This repository was archived by the owner on Jul 24, 2024. It is now read-only.
File tree Expand file tree Collapse file tree 1 file changed +24
-0
lines changed Expand file tree Collapse file tree 1 file changed +24
-0
lines changed Original file line number Diff line number Diff line change @@ -703,6 +703,30 @@ lemma le_mul_of_one_le_left' [mul_pos_mono α] (h : 1 ≤ a) (b0 : 0 ≤ b) :
703
703
b ≤ a * b :=
704
704
le_mul_of_one_le_of_le' h le_rfl b0
705
705
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
+
706
730
end partial_order
707
731
708
732
section linear_order
You can’t perform that action at this time.
0 commit comments