Idris2/tests/idris2/basic019/expected
2020-08-18 19:25:36 +01:00

9 lines
409 B
Plaintext

1/1: Building CaseBlock (CaseBlock.idr)
Main> Main.foo : (x : Nat) -> (case x of {0 => Nat -> Nat; S k => Nat})
Main> Prelude.elem : Eq a => a -> List a -> Bool
elem x [] = False
elem x (y :: ys) = (x == y) || Delay (elem x ys)
Main> PrimIO.io_bind : (1 _ : IO a) -> (1 _ : (a -> IO b)) -> IO b
io_bind (MkIO fn) k = MkIO (\1 w => let MkIORes x' w' = fn w in let MkIO res = k x' in res w')
Main> Bye for now!