lean2/tests/lean/run/e1.lean

16 lines
328 B
Text

prelude
definition Prop : Type.{1} := Type.{0}
constant eq : forall {A : Type}, A → A → Prop
constant N : Type.{1}
constants a b c : N
infix `=`:50 := eq
check a = b
constant f : Prop → N → N
constant g : N → N → N
precedence `+`:50
infixl + := f
infixl + := g
check a + b + c
constant p : Prop
check p + a + b + c