mirror of
https://github.com/idris-lang/Idris2.git
synced 2024-12-18 00:31:57 +03:00
8291c8bbeb
Should have done this ages ago, it was much easier than I expected... this adds an explicit error clause before running the pattern match compiler for runtime case trees, but only if the coverage checker finds there are missing cases.
25 lines
521 B
Idris
25 lines
521 B
Idris
foo : Maybe a -> a
|
|
foo (Just x) = x
|
|
|
|
data Vect : ? -> Type -> Type where
|
|
Nil : Vect Z a
|
|
(::) : a -> Vect k a -> Vect (S k) a
|
|
|
|
data Fin : Nat -> Type where
|
|
FZ : Fin (S k)
|
|
FS : Fin k -> Fin (S k)
|
|
|
|
lookup : Fin n -> Vect n a -> a
|
|
lookup FZ (x :: xs) = x
|
|
lookup (FS k) (x :: xs) = lookup k xs
|
|
|
|
lookup' : Fin n -> Vect n a -> a
|
|
lookup' (FS k) (x :: xs) = lookup' k xs
|
|
|
|
lookup'' : Fin n -> Vect n a -> a
|
|
lookup'' n xs = lookup' n xs
|
|
|
|
main : IO ()
|
|
main = do let x = foo Nothing
|
|
printLn (the Int x)
|