7 lines
117 B
Text
7 lines
117 B
Text
|
Definition B : Type := Bool
|
||
|
Definition T : Type 1 := Type
|
||
|
Variable N : T
|
||
|
Variable x : N
|
||
|
Variable a : B
|
||
|
Axiom H : a
|