Skip to content

Commit e6628dd

Browse files
authored
feat: Match mathlib#16761 (#840)
* feat: Match mathlib#16761 * fix
1 parent 8aaf280 commit e6628dd

File tree

1 file changed

+10
-0
lines changed

1 file changed

+10
-0
lines changed

Mathlib/Algebra/Order/Monoid/Lemmas.lean

Lines changed: 10 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -940,6 +940,16 @@ theorem mul_eq_one_iff' [CovariantClass α α (· * ·) (· ≤ ·)]
940940
-- `fun ⟨ha', hb'⟩ => by rw [ha', hb', mul_one]`,
941941
-- had its `to_additive`-ization fail due to some bug
942942

943+
@[to_additive] lemma mul_le_mul_iff_of_ge [CovariantClass α α (· * ·) (· ≤ ·)]
944+
[CovariantClass α α (swap (· * ·)) (· ≤ ·)] [CovariantClass α α (· * ·) (· < ·)]
945+
[CovariantClass α α (swap (· * ·)) (· < ·)] {a₁ a₂ b₁ b₂ : α} (ha : a₁ ≤ a₂) (hb : b₁ ≤ b₂) :
946+
a₂ * b₂ ≤ a₁ * b₁ ↔ a₁ = a₂ ∧ b₁ = b₂ := by
947+
refine' ⟨fun h ↦ _, by rintro ⟨rfl, rfl⟩; rfl⟩
948+
simp only [eq_iff_le_not_lt, ha, hb, true_and]
949+
refine' ⟨fun ha ↦ h.not_lt _, fun hb ↦ h.not_lt _⟩
950+
{ exact mul_lt_mul_of_lt_of_le ha hb }
951+
{ exact mul_lt_mul_of_le_of_lt ha hb }
952+
943953
section Left
944954

945955
variable [CovariantClass α α (· * ·) (· ≤ ·)] {a b : α}

0 commit comments

Comments
 (0)