Idris2/tests/idris2/with003/Main.idr
2020-05-22 20:26:10 +02:00

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