Idris2/tests/idris2/positivity002/Issue660.idr
Guillaume ALLAIS 7ccc47712e [ re #1087 ] Better error messages in the REPL
(as well as in type signatures now that I know how to do that)
2021-02-19 12:34:19 +00:00

16 lines
239 B
Idris

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
%logging off
data E : Type where