Idris2/tests/idris2/total/total015/CoveringData.idr
2023-09-07 14:57:22 +01:00

13 lines
234 B
Idris

%default total
data Tree a = Node a (Tree a) (Tree a)
failing "Nope is not total, not strictly positive"
data Nope : Type where
MkNope : Tree (Not Nope) -> Nope
covering
data Yep : Type where
MkYep : Tree (Not Yep) -> Yep