Idris2/tests/idris2/positivity001/Issue660.idr

9 lines
152 B
Idris
Raw Normal View History

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