lean2/tests/lean/run/n3.lean
Leonardo de Moura 5eaf04518b refactor(*): rename Bool to Prop
Signed-off-by: Leonardo de Moura <leonardo@microsoft.com>
2014-07-22 09:43:18 -07:00

22 lines
616 B
Text

definition Prop [inline] : Type.{1} := Type.{0}
variable N : Type.{1}
variable and : Prop → Prop → Prop
infixr `∧`:35 := and
variable le : N → N → Prop
variable lt : N → N → Prop
variable f : N → N
variable add : N → N → N
infixl `+`:65 := add
precedence `≤`:50
precedence `<`:50
infixl ≤ := le
infixl < := lt
notation A ≤ B:prev ≤ C:prev := A ≤ B ∧ B ≤ C
notation A ≤ B:prev < C:prev := A ≤ B ∧ B < C
notation A < B:prev ≤ C:prev := A < B ∧ B ≤ C
variables a b c d e : N
check a ≤ b ≤ f c + b ∧ a < b
check a ≤ d
check a < b ≤ c
check a ≤ b < c
check a < b