Skip to content

Commit

Permalink
feat(algebra/order/field): lemmas relating a / b and a when `1 ≤ …
Browse files Browse the repository at this point in the history
…b` and `1 < b` (#11333)

This PR is a collection of items that #7891 adds in and that aren't declared on `master` yet. Please let me know if I overlooked something.

After merging it, #7891 can theoretically be closed.



Co-authored-by: Benjamin Davidson <68528197+benjamindavidson@users.noreply.github.com>
  • Loading branch information
arthurpaulino and benjamindavidson committed Jan 11, 2022
1 parent 2865d8c commit eb9c152
Showing 1 changed file with 7 additions and 1 deletion.
8 changes: 7 additions & 1 deletion src/algebra/order/field.lean
Expand Up @@ -395,13 +395,19 @@ lemma div_lt_div' (hac : a ≤ c) (hbd : d < b) (c0 : 0 < c) (d0 : 0 < d) :
a / b < c / d :=
(div_lt_div_iff (d0.trans hbd) d0).2 (mul_lt_mul' hac hbd d0.le c0)

lemma div_lt_div_of_lt_left (hb : 0 < b) (h : b < a) (hc : 0 < c) : c / a < c / b :=
lemma div_lt_div_of_lt_left (hc : 0 < c) (hb : 0 < b) (h : b < a) : c / a < c / b :=
(div_lt_div_left hc (hb.trans h) hb).mpr h

/-!
### Relating one division and involving `1`
-/

lemma div_le_self (ha : 0 ≤ a) (hb : 1 ≤ b) : a / b ≤ a :=
by simpa only [div_one] using div_le_div_of_le_left ha zero_lt_one hb

lemma div_lt_self (ha : 0 < a) (hb : 1 < b) : a / b < a :=
by simpa only [div_one] using div_lt_div_of_lt_left ha zero_lt_one hb

lemma one_le_div (hb : 0 < b) : 1 ≤ a / b ↔ b ≤ a :=
by rw [le_div_iff hb, one_mul]

Expand Down

0 comments on commit eb9c152

Please sign in to comment.