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

Commit 1675b78

Browse files
committed
feat(algebra/order/monoid_lemmas_zero_lt): add some lemmas assuming mul_zero_one_class partial_order (#13375)
1 parent 95413e2 commit 1675b78

File tree

1 file changed

+24
-0
lines changed

1 file changed

+24
-0
lines changed

src/algebra/order/monoid_lemmas_zero_lt.lean

Lines changed: 24 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -703,6 +703,30 @@ lemma le_mul_of_one_le_left' [mul_pos_mono α] (h : 1 ≤ a) (b0 : 0 ≤ b) :
703703
b ≤ a * b :=
704704
le_mul_of_one_le_of_le' h le_rfl b0
705705

706+
lemma le_of_mul_le_of_one_le_left' [pos_mul_mono α]
707+
(h : a * b ≤ c) (hle : 1 ≤ b) (a0 : 0 ≤ a) :
708+
a ≤ c :=
709+
a0.lt_or_eq.elim (le_of_mul_le_of_one_le_left h hle)
710+
(λ ha, by simpa only [← ha, zero_mul] using h)
711+
712+
lemma le_of_le_mul_of_le_one_left' [pos_mul_mono α]
713+
(h : a ≤ b * c) (hle : c ≤ 1) (b0 : 0 ≤ b) :
714+
a ≤ b :=
715+
b0.lt_or_eq.elim (le_of_le_mul_of_le_one_left h hle)
716+
(λ hb, by simpa only [← hb, zero_mul] using h)
717+
718+
lemma le_of_mul_le_of_one_le_right' [mul_pos_mono α]
719+
(h : a * b ≤ c) (hle : 1 ≤ a) (b0 : 0 ≤ b) :
720+
b ≤ c :=
721+
b0.lt_or_eq.elim (le_of_mul_le_of_one_le_right h hle)
722+
(λ ha, by simpa only [← ha, mul_zero] using h)
723+
724+
lemma le_of_le_mul_of_le_one_right' [mul_pos_mono α]
725+
(h : a ≤ b * c) (hle : b ≤ 1) (c0 : 0 ≤ c) :
726+
a ≤ c :=
727+
c0.lt_or_eq.elim (le_of_le_mul_of_le_one_right h hle)
728+
(λ ha, by simpa only [← ha, mul_zero] using h)
729+
706730
end partial_order
707731

708732
section linear_order

0 commit comments

Comments
 (0)