Idris2/tests/idris2/basic031/erased.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
377 B
Idris

data MyMaybe : (0 x : Type) -> Type where
MyNothing : MyMaybe a
MyJust : a -> MyMaybe a
-- Should fail since type argument is deleted
nameOf : Type -> String
nameOf (MyMaybe Bool) = "MyMaybe Bool"
nameOf (MyMaybe Int) = "MyMaybe Int"
nameOf _ = "Unknown"
main : IO ()
main = do
putStrLn (nameOf (MyMaybe Bool))
putStrLn (nameOf (MyMaybe Int))
putStrLn (nameOf Int)