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

Commit 384c9be

Browse files
jdsalchowmergify[bot]
authored andcommitted
feat (analysis/normed_space/basic.lean): implement reverse triangle inequality (#831)
* implement reverse triangle inequality * make parameters explicit
1 parent 07aa1e3 commit 384c9be

File tree

1 file changed

+9
-0
lines changed

1 file changed

+9
-0
lines changed

src/analysis/normed_space/basic.lean

Lines changed: 9 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -87,6 +87,15 @@ calc ∥-g∥ = ∥0 - g∥ : by simp
8787
... = ∥g - 0∥ : (dist_eq_norm g 0)
8888
... = ∥g∥ : by simp
8989

90+
lemma norm_reverse_triangle' (a b : α) : ∥a∥ - ∥b∥ ≤ ∥a - b∥ :=
91+
by simpa using add_le_add (norm_triangle (a - b) (b)) (le_refl (-∥b∥))
92+
93+
lemma norm_reverse_triangle (a b : α) : abs(∥a∥ - ∥b∥) ≤ ∥a - b∥ :=
94+
suffices -(∥a∥ - ∥b∥) ≤ ∥a - b∥, from abs_le_of_le_of_neg_le (norm_reverse_triangle' a b) this,
95+
calc -(∥a∥ - ∥b∥) = ∥b∥ - ∥a∥ : by abel
96+
... ≤ ∥b - a∥ : norm_reverse_triangle' b a
97+
... = ∥a - b∥ : by rw ← norm_neg (a - b); simp
98+
9099
lemma norm_triangle_sub {a b : α} : ∥a - b∥ ≤ ∥a∥ + ∥b∥ :=
91100
by simpa only [sub_eq_add_neg, norm_neg] using norm_triangle a (-b)
92101

0 commit comments

Comments
 (0)