Idris2/tests/idris2/misc/with003/Main.idr
2023-09-07 14:57:22 +01:00

15 lines
288 B
Idris

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