Idris2/tests/idris2/positivity001/Issue660.idr
2020-09-14 18:37:47 +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 ()