Idris2/tests/idris2/positivity002/Issue660.idr

12 lines
202 B
Idris
Raw Normal View History

module Issue660
%default total
%logging declare.data.parameters 20
data C : Type -> Type where
MkC : List a -> C a
data D : Type -> Type where
MkD : {0 a : Type} -> let 0 b = List a in b -> D a