Zulip Chat Archive
Stream: Is there code for X?
Topic: two_le_add_inv
Rémy Degenne (Oct 05 2021 at 15:18):
Do we have this?
lemma two_le_add_inv {x : ℝ} (hx : 0 < x) : 2 ≤ x + x⁻¹ := sorry
Chris Hughes (Oct 05 2021 at 15:26):
lemma two_le_add_inv {x : ℝ} (hx : 0 < x) : 2 ≤ x + x⁻¹ :=
le_of_mul_le_mul_left
(sub_nonneg.1 $
calc 0 ≤ (x - 1) ^ 2 : pow_two_nonneg _
... = _ : by field_simp [ne_of_gt hx]; ring)
hx
Rémy Degenne (Oct 05 2021 at 15:28):
That's three lines shorter than mine :) Thanks.
Should I add it, if that exact statement is not already somewhere under another name?
Rémy Degenne (Oct 05 2021 at 15:31):
I guess that yes, I want to add it if it does not already exist. My original question was more "does it exist already in a place I did not find?", and not really "how do I prove this?".
Alex J. Best (Oct 05 2021 at 15:38):
Maybe it should go in analysis.mean_inequalities? its sortof a special case of AM-GM?
Patrick Massot (Oct 05 2021 at 15:41):
This has nothing to do with real or complex numbers so it should probably not go in analysis
Patrick Massot (Oct 05 2021 at 15:42):
It should assume a linear order field or something like this
Yury G. Kudryashov (Oct 05 2021 at 15:56):
Should we have AM-GM for linear ordered fields (with pow
instead of root)?
Last updated: Dec 20 2023 at 11:08 UTC