Skip to content
This repository was archived by the owner on Jul 24, 2024. It is now read-only.

Commit b9354dd

Browse files
committed
feat(algebra/ordered_ring): a product is at least one if both factors are (#6172)
Add single lemma one_le_mul_of_one_le_of_one_le The lemma is stated for an `ordered_semiring`, but only multiplication is used. There does not seem to be an `ordered_monoid` class where this lemma would fit. Relevant Zulip chat: https://leanprover.zulipchat.com/#narrow/stream/113489-new-members/topic/ordered_monoid.3F
1 parent 194ec66 commit b9354dd

File tree

1 file changed

+4
-0
lines changed

1 file changed

+4
-0
lines changed

src/algebra/ordered_ring.lean

Lines changed: 4 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -144,6 +144,10 @@ calc a + (2 + b) ≤ a + (a + a * b) :
144144
add_le_add_left (add_le_add a2 (le_mul_of_one_le_left b0 (one_le_two.trans a2))) a
145145
... ≤ a * (2 + b) : by rw [mul_add, mul_two, add_assoc]
146146

147+
lemma one_le_mul_of_one_le_of_one_le {a b : α} (a1 : 1 ≤ a) (b1 : 1 ≤ b) :
148+
(1 : α) ≤ a * b :=
149+
(mul_one (1 : α)).symm.le.trans (mul_le_mul a1 b1 zero_le_one (zero_le_one.trans a1))
150+
147151
section
148152
variable [nontrivial α]
149153

0 commit comments

Comments
 (0)