Idris2/tests/idris2/with003/Main.idr
Edwin Brady d12487f529 HasIO interface for IO actions
Also updates the Prelude and some base libraries to use HasIO rather
than using IO directly.
2020-06-21 01:18:43 +01:00

15 lines
289 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 a -> IO b -> IO b
(>>=) f x = f *> x