mirror of
https://github.com/idris-lang/Idris2.git
synced 2024-12-17 08:11:45 +03:00
16 lines
377 B
Idris
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)
|