lean2/tests/lean/run/t1.lean

10 lines
325 B
Text

prelude
definition Prop : Type.{1} := Type.{0}
print raw ((Prop))
print raw Prop
print raw fun (x y : Prop), x x
print raw fun (x y : Prop) {z : Prop}, x y
print raw λ [x y : Prop] {z : Prop}, x z
print raw Pi (x y : Prop) {z : Prop}, x
print raw ∀ (x y : Prop) {z : Prop}, x
print raw forall {x y : Prop} w {z : Prop}, x