Skip to content

Commit c8818ba

Browse files
committed
feat(NormedSpace/Basic): add dist_smul_add_one_sub_smul_le (#9982)
From sphere-eversion (slightly golfed); I'm just upstreaming it.
1 parent ca91ff1 commit c8818ba

File tree

1 file changed

+11
-0
lines changed

1 file changed

+11
-0
lines changed

Mathlib/Analysis/NormedSpace/Basic.lean

Lines changed: 11 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -86,6 +86,17 @@ variable {E : Type*} [SeminormedAddCommGroup E] [NormedSpace α E]
8686

8787
variable {F : Type*} [SeminormedAddCommGroup F] [NormedSpace α F]
8888

89+
theorem dist_smul_add_one_sub_smul_le [NormedSpace ℝ E] {r : ℝ} {x y : E} (h : r ∈ Icc 0 1) :
90+
dist (r • x + (1 - r) • y) x ≤ dist y x :=
91+
calc
92+
dist (r • x + (1 - r) • y) x = ‖1 - r‖ * ‖x - y‖ := by
93+
simp_rw [dist_eq_norm', ← norm_smul, sub_smul, one_smul, smul_sub, ← sub_sub, ← sub_add,
94+
sub_right_comm]
95+
_ = (1 - r) * dist y x := by
96+
rw [Real.norm_eq_abs, abs_eq_self.mpr (sub_nonneg.mpr h.2), dist_eq_norm']
97+
_ ≤ (1 - 0) * dist y x := by gcongr; exact h.1
98+
_ = dist y x := by rw [sub_zero, one_mul]
99+
89100
theorem eventually_nhds_norm_smul_sub_lt (c : α) (x : E) {ε : ℝ} (h : 0 < ε) :
90101
∀ᶠ y in 𝓝 x, ‖c • (y - x)‖ < ε :=
91102
have : Tendsto (fun y => ‖c • (y - x)‖) (𝓝 x) (𝓝 0) :=

0 commit comments

Comments
 (0)