mirror of
https://github.com/idris-lang/Idris2.git
synced 2024-12-19 09:12:34 +03:00
8 lines
373 B
Plaintext
8 lines
373 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 : Foldable t => Eq a => a -> t a -> Bool
|
|
elem = elemBy ==
|
|
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!
|