mirror of
https://github.com/idris-lang/Idris2.git
synced 2024-12-16 07:34:45 +03:00
d12487f529
Also updates the Prelude and some base libraries to use HasIO rather than using IO directly.
15 lines
289 B
Idris
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
|