2014-07-22 16:43:18 +00:00
|
|
|
definition Prop [inline] : Type.{1} := Type.{0}
|
|
|
|
variable eq : forall {A : Type}, A → A → Prop
|
2014-06-25 15:30:09 +00:00
|
|
|
variable N : Type.{1}
|
|
|
|
variables a b c : N
|
2014-07-01 23:55:41 +00:00
|
|
|
infix `=`:50 := eq
|
2014-06-25 15:30:09 +00:00
|
|
|
check a = b
|
|
|
|
|
2014-07-22 16:43:18 +00:00
|
|
|
variable f : Prop → N → N
|
2014-06-25 15:30:09 +00:00
|
|
|
variable g : N → N → N
|
|
|
|
precedence `+`:50
|
|
|
|
infixl + := f
|
|
|
|
infixl + := g
|
|
|
|
check a + b + c
|
2014-07-22 16:43:18 +00:00
|
|
|
variable p : Prop
|
2014-06-25 15:30:09 +00:00
|
|
|
check p + a + b + c
|