Idris2/tests/idris2/coverage003/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

18 lines
243 B
Idris

%default partial
foo : (Nat, Nat) -> Nat
foo (Z, Z) = Z
bar : {a : _} -> a -> Nat
bar Z = Z
bar (S _) = S Z
cty : (a : Type) -> a -> Nat
cty Nat Z = Z
cty Nat (S _) = S Z
cty _ x = S (S Z)
badBar : a -> Nat
badBar Z = Z
badBar (S _) = S Z