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

9 lines
152 B
Idris

module Issue660
%default total
data Sig : (a : Type) -> (a -> Type) -> Type where
data Value : Unit -> Type where
MkV : Sig Unit Value -> Value ()