Idris2/tests/idris2/with003/Main.idr

15 lines
288 B
Idris
Raw Normal View History

2020-05-22 21:26:10 +03:00
module Main
import Data.List
import Data.Vect
-- needs to be concretely in IO to test error messages
myPrintLn : String -> IO ()
myPrintLn = printLn
2020-05-22 21:26:10 +03:00
-- add some definition of (>>=) in another namespace
namespace Other
public export
(>>) : IO () -> IO b -> IO b
(>>) f x = f *> x