Idris2/tests/idris2/basic007/DoLocal.idr
Edwin Brady a972778eab Add test script
They don't all pass yet, for minor reasons. Coming shortly...
Unfortunately the startup overhead for chez is really noticeable here!
2020-05-19 18:25:18 +01:00

16 lines
414 B
Idris

import Stuff
(>>=) : (Maybe a) -> (a -> Maybe b) -> Maybe b
(>>=) Nothing k = Nothing
(>>=) (Just x) k = k x
mthings : (foo : Maybe (Maybe Int)) -> (bar : Maybe (Maybe Int)) -> Maybe Int
mthings mx my
= do Just x <- mx
| Nothing => Just 0
Just y <- my
| Nothing => Just 1
let z : Int -> Int
z x = prim__add_Int x y
Just (z (prim__add_Int x x))