Documentation

Mathlib.Init.Data.Int.Order

The order relation on the integers #

theorem Int.le.elim {a : } {b : } (h : a b) {P : Prop} (h' : ∀ (n : ), a + n = bP) :
P
theorem Int.le_of_ofNat_le_ofNat {m : } {n : } :
m nm n

Alias of the forward direction of Int.ofNat_le.

theorem Int.ofNat_le_ofNat_of_le {m : } {n : } :
m nm n

Alias of the reverse direction of Int.ofNat_le.

theorem Int.lt.elim {a : } {b : } (h : a < b) {P : Prop} (h' : ∀ (n : ), a + (Nat.succ n) = bP) :
P
theorem Int.ofNat_lt_ofNat_of_lt {n : } {m : } :
n < mn < m

Alias of the reverse direction of Int.ofNat_lt.

theorem Int.lt_of_ofNat_lt_ofNat {n : } {m : } :
n < mn < m

Alias of the forward direction of Int.ofNat_lt.

theorem Int.neg_mul_eq_neg_mul_symm (a : ) (b : ) :
-a * b = -(a * b)
theorem Int.mul_neg_eq_neg_mul_symm (a : ) (b : ) :
a * -b = -(a * b)
theorem Int.eq_zero_or_eq_zero_of_mul_eq_zero {a : } {b : } (h : a * b = 0) :
a = 0 b = 0