Idris2/tests/idris2/coverage004/Cover.idr
Edwin Brady 498421a236 All functions now need to be covering by default
This has caught a couple of things in the Idris 2 code base itself. Some
tests needed partial annotations too.
2020-05-24 19:58:20 +01:00

15 lines
256 B
Idris

%default partial
data Foo : Type -> Type where
IsNat : Foo Nat
IsBool : Foo Bool
okay : a -> Foo a -> Bool
okay Z IsNat = False
okay True IsBool = True
bad : a -> Foo a -> Bool
bad Z IsNat = False
bad True IsBool = True
bad (Just 0) _ = False