4946f55290
Signed-off-by: Leonardo de Moura <leonardo@microsoft.com>
15 lines
320 B
Text
15 lines
320 B
Text
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
|