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

Commit d5344df

Browse files
committed
feat(algebra/order/ring): lt_mul_{left,right,self} (#15848)
1 parent d1795d6 commit d5344df

File tree

1 file changed

+9
-0
lines changed

1 file changed

+9
-0
lines changed

src/algebra/order/ring.lean

Lines changed: 9 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -366,6 +366,15 @@ by classical; exact decidable.lt_mul_of_one_lt_left
366366
lemma lt_two_mul_self [nontrivial α] (ha : 0 < a) : a < 2 * a :=
367367
lt_mul_of_one_lt_left ha one_lt_two
368368

369+
lemma lt_mul_left (hn : 0 < a) (hm : 1 < b) : a < b * a :=
370+
by { convert mul_lt_mul_of_pos_right hm hn, rw one_mul }
371+
372+
lemma lt_mul_right (hn : 0 < a) (hm : 1 < b) : a < a * b :=
373+
by { convert mul_lt_mul_of_pos_left hm hn, rw mul_one }
374+
375+
lemma lt_mul_self (hn : 1 < a) : a < a * a :=
376+
lt_mul_left (hn.trans_le' zero_le_one) hn
377+
369378
-- See Note [decidable namespace]
370379
protected lemma decidable.add_le_mul_two_add [@decidable_rel α (≤)] {a b : α}
371380
(a2 : 2 ≤ a) (b0 : 0 ≤ b) : a + (2 + b) ≤ a * (2 + b) :=

0 commit comments

Comments
 (0)