mirror of
https://github.com/idris-lang/Idris2.git
synced 2024-12-15 14:23:32 +03:00
15 lines
288 B
Idris
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
|