lean2/tests/lean/ty2.lean
Leonardo de Moura 390f7eaec8 test(kernel/typechecker): type checker
Signed-off-by: Leonardo de Moura <leonardo@microsoft.com>
2013-11-16 15:01:39 -08:00

6 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