Idris2/tests/idris2/linear016/Issue2895_2.idr

16 lines
241 B
Idris
Raw Normal View History

2023-02-25 15:19:29 +03:00
record Ty where
constructor MkTy
0 obj : Type
record TyProj (d: Ty) where
constructor MkTyProj
proj : d.obj
DepLensToDepOptic :
{c1 : TyProj (MkTy (Nat -> Type))} ->
(c1.proj 3) ->
Type
DepLensToDepOptic =
(\(b) => ?mmm)