Idris2/tests/idris2/reflection/reflection017/StillCantEscape.idr
2023-09-07 14:57:22 +01:00

14 lines
226 B
Idris

module StillCantEscape
import CanElabType
import Language.Reflection
%language ElabReflection
-- check that zero does not leak, should not typecheck
failing "CanElabType.T is private"
T' : Type
T' = %runElab elabExpr