Idris2/tests/idris2/linear/linear016/Issue2895_2.idr
2023-09-07 14:57:22 +01:00

16 lines
241 B
Idris

record Ty where
constructor MkTy
0 obj : Type
record TyProj (d: Ty) where
constructor MkTyProj
proj : d.obj
DepLensToDepOptic :
{c1 : TyProj (MkTy (Nat -> Type))} ->
(proj c1 3) ->
Type
DepLensToDepOptic =
(\(b) => ?mmm)