mirror of
https://github.com/idris-lang/Idris2.git
synced 2024-12-18 16:51:51 +03:00
11 lines
185 B
Idris
11 lines
185 B
Idris
module Main
|
|
|
|
import Data.List
|
|
import Data.Vect
|
|
|
|
-- add some definition of (>>=) in another namespace
|
|
namespace Other
|
|
public export
|
|
(>>=) : IO a -> IO b -> IO b
|
|
(>>=) f x = f *> x
|