lean2/tests/lean/ty2.lean

7 lines
117 B
Text
Raw Normal View History

Definition B : Type := Bool
Definition T : Type 1 := Type
Variable N : T
Variable x : N
Variable a : B
Axiom H : a