mirror of
https://github.com/idris-lang/Idris2.git
synced 2024-12-15 14:23:32 +03:00
7ccc47712e
(as well as in type signatures now that I know how to do that)
16 lines
239 B
Idris
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
|