Documentation

Mathlib.Analysis.NormedSpace.Pointwise

Properties of pointwise scalar multiplication of sets in normed spaces. #

We explore the relationships between scalar multiplication of sets in vector spaces, and the norm. Notably, we express arbitrary balls as rescaling of other balls, and we show that the multiplication of bounded sets remain bounded.

theorem ediam_smul_le {𝕜 : Type u_1} {E : Type u_2} [SeminormedAddCommGroup 𝕜] [SeminormedAddCommGroup E] [SMulZeroClass 𝕜 E] [BoundedSMul 𝕜 E] (c : 𝕜) (s : Set E) :
theorem ediam_smul₀ {𝕜 : Type u_1} {E : Type u_2} [NormedDivisionRing 𝕜] [SeminormedAddCommGroup E] [Module 𝕜 E] [BoundedSMul 𝕜 E] (c : 𝕜) (s : Set E) :
theorem diam_smul₀ {𝕜 : Type u_1} {E : Type u_2} [NormedDivisionRing 𝕜] [SeminormedAddCommGroup E] [Module 𝕜 E] [BoundedSMul 𝕜 E] (c : 𝕜) (x : Set E) :
theorem infEdist_smul₀ {𝕜 : Type u_1} {E : Type u_2} [NormedDivisionRing 𝕜] [SeminormedAddCommGroup E] [Module 𝕜 E] [BoundedSMul 𝕜 E] {c : 𝕜} (hc : c 0) (s : Set E) (x : E) :
theorem infDist_smul₀ {𝕜 : Type u_1} {E : Type u_2} [NormedDivisionRing 𝕜] [SeminormedAddCommGroup E] [Module 𝕜 E] [BoundedSMul 𝕜 E] {c : 𝕜} (hc : c 0) (s : Set E) (x : E) :
theorem smul_ball {𝕜 : Type u_1} {E : Type u_2} [NormedField 𝕜] [SeminormedAddCommGroup E] [NormedSpace 𝕜 E] {c : 𝕜} (hc : c 0) (x : E) (r : ) :
theorem smul_unitBall {𝕜 : Type u_1} {E : Type u_2} [NormedField 𝕜] [SeminormedAddCommGroup E] [NormedSpace 𝕜 E] {c : 𝕜} (hc : c 0) :
theorem smul_sphere' {𝕜 : Type u_1} {E : Type u_2} [NormedField 𝕜] [SeminormedAddCommGroup E] [NormedSpace 𝕜 E] {c : 𝕜} (hc : c 0) (x : E) (r : ) :
theorem smul_closedBall' {𝕜 : Type u_1} {E : Type u_2} [NormedField 𝕜] [SeminormedAddCommGroup E] [NormedSpace 𝕜 E] {c : 𝕜} (hc : c 0) (x : E) (r : ) :
theorem set_smul_sphere_zero {𝕜 : Type u_1} {E : Type u_2} [NormedField 𝕜] [SeminormedAddCommGroup E] [NormedSpace 𝕜 E] {s : Set 𝕜} (hs : 0s) (r : ) :
s Metric.sphere 0 r = (fun (x : E) => x) ⁻¹' ((fun (x : 𝕜) => x * r) '' s)
theorem Bornology.IsBounded.smul₀ {𝕜 : Type u_1} {E : Type u_2} [NormedField 𝕜] [SeminormedAddCommGroup E] [NormedSpace 𝕜 E] {s : Set E} (hs : Bornology.IsBounded s) (c : 𝕜) :

Image of a bounded set in a normed space under scalar multiplication by a constant is bounded. See also Bornology.IsBounded.smul for a similar lemma about an isometric action.

theorem eventually_singleton_add_smul_subset {𝕜 : Type u_1} {E : Type u_2} [NormedField 𝕜] [SeminormedAddCommGroup E] [NormedSpace 𝕜 E] {x : E} {s : Set E} (hs : Bornology.IsBounded s) {u : Set E} (hu : u nhds x) :
∀ᶠ (r : 𝕜) in nhds 0, {x} + r s u

If s is a bounded set, then for small enough r, the set {x} + r • s is contained in any fixed neighborhood of x.

theorem smul_unitBall_of_pos {E : Type u_2} [SeminormedAddCommGroup E] [NormedSpace E] {r : } (hr : 0 < r) :

In a real normed space, the image of the unit ball under scalar multiplication by a positive constant r is the ball of radius r.

theorem Ioo_smul_sphere_zero {E : Type u_2} [SeminormedAddCommGroup E] [NormedSpace E] {a : } {b : } {r : } (ha : 0 a) (hr : 0 < r) :
theorem exists_dist_eq {E : Type u_2} [SeminormedAddCommGroup E] [NormedSpace E] (x : E) (z : E) {a : } {b : } (ha : 0 a) (hb : 0 b) (hab : a + b = 1) :
∃ (y : E), dist x y = b * dist x z dist y z = a * dist x z
theorem exists_dist_le_le {E : Type u_2} [SeminormedAddCommGroup E] [NormedSpace E] {x : E} {z : E} {δ : } {ε : } (hδ : 0 δ) (hε : 0 ε) (h : dist x z ε + δ) :
∃ (y : E), dist x y δ dist y z ε
theorem exists_dist_le_lt {E : Type u_2} [SeminormedAddCommGroup E] [NormedSpace E] {x : E} {z : E} {δ : } {ε : } (hδ : 0 δ) (hε : 0 < ε) (h : dist x z < ε + δ) :
∃ (y : E), dist x y δ dist y z < ε
theorem exists_dist_lt_le {E : Type u_2} [SeminormedAddCommGroup E] [NormedSpace E] {x : E} {z : E} {δ : } {ε : } (hδ : 0 < δ) (hε : 0 ε) (h : dist x z < ε + δ) :
∃ (y : E), dist x y < δ dist y z ε
theorem exists_dist_lt_lt {E : Type u_2} [SeminormedAddCommGroup E] [NormedSpace E] {x : E} {z : E} {δ : } {ε : } (hδ : 0 < δ) (hε : 0 < ε) (h : dist x z < ε + δ) :
∃ (y : E), dist x y < δ dist y z < ε
theorem disjoint_ball_ball_iff {E : Type u_2} [SeminormedAddCommGroup E] [NormedSpace E] {x : E} {y : E} {δ : } {ε : } (hδ : 0 < δ) (hε : 0 < ε) :
Disjoint (Metric.ball x δ) (Metric.ball y ε) δ + ε dist x y
theorem disjoint_ball_closedBall_iff {E : Type u_2} [SeminormedAddCommGroup E] [NormedSpace E] {x : E} {y : E} {δ : } {ε : } (hδ : 0 < δ) (hε : 0 ε) :
theorem disjoint_closedBall_ball_iff {E : Type u_2} [SeminormedAddCommGroup E] [NormedSpace E] {x : E} {y : E} {δ : } {ε : } (hδ : 0 δ) (hε : 0 < ε) :
theorem disjoint_closedBall_closedBall_iff {E : Type u_2} [SeminormedAddCommGroup E] [NormedSpace E] {x : E} {y : E} {δ : } {ε : } (hδ : 0 δ) (hε : 0 ε) :
@[simp]
theorem infEdist_thickening {E : Type u_2} [SeminormedAddCommGroup E] [NormedSpace E] {δ : } (hδ : 0 < δ) (s : Set E) (x : E) :
@[simp]
theorem thickening_thickening {E : Type u_2} [SeminormedAddCommGroup E] [NormedSpace E] {δ : } {ε : } (hε : 0 < ε) (hδ : 0 < δ) (s : Set E) :
@[simp]
theorem cthickening_thickening {E : Type u_2} [SeminormedAddCommGroup E] [NormedSpace E] {δ : } {ε : } (hε : 0 ε) (hδ : 0 < δ) (s : Set E) :
@[simp]
theorem closure_thickening {E : Type u_2} [SeminormedAddCommGroup E] [NormedSpace E] {δ : } (hδ : 0 < δ) (s : Set E) :
@[simp]
theorem thickening_cthickening {E : Type u_2} [SeminormedAddCommGroup E] [NormedSpace E] {δ : } {ε : } (hε : 0 < ε) (hδ : 0 δ) (s : Set E) :
@[simp]
theorem cthickening_cthickening {E : Type u_2} [SeminormedAddCommGroup E] [NormedSpace E] {δ : } {ε : } (hε : 0 ε) (hδ : 0 δ) (s : Set E) :
@[simp]
theorem thickening_ball {E : Type u_2} [SeminormedAddCommGroup E] [NormedSpace E] {δ : } {ε : } (hε : 0 < ε) (hδ : 0 < δ) (x : E) :
@[simp]
theorem thickening_closedBall {E : Type u_2} [SeminormedAddCommGroup E] [NormedSpace E] {δ : } {ε : } (hε : 0 < ε) (hδ : 0 δ) (x : E) :
@[simp]
theorem cthickening_ball {E : Type u_2} [SeminormedAddCommGroup E] [NormedSpace E] {δ : } {ε : } (hε : 0 ε) (hδ : 0 < δ) (x : E) :
@[simp]
theorem cthickening_closedBall {E : Type u_2} [SeminormedAddCommGroup E] [NormedSpace E] {δ : } {ε : } (hε : 0 ε) (hδ : 0 δ) (x : E) :
theorem ball_add_ball {E : Type u_2} [SeminormedAddCommGroup E] [NormedSpace E] {δ : } {ε : } (hε : 0 < ε) (hδ : 0 < δ) (a : E) (b : E) :
Metric.ball a ε + Metric.ball b δ = Metric.ball (a + b) (ε + δ)
theorem ball_sub_ball {E : Type u_2} [SeminormedAddCommGroup E] [NormedSpace E] {δ : } {ε : } (hε : 0 < ε) (hδ : 0 < δ) (a : E) (b : E) :
Metric.ball a ε - Metric.ball b δ = Metric.ball (a - b) (ε + δ)
theorem ball_add_closedBall {E : Type u_2} [SeminormedAddCommGroup E] [NormedSpace E] {δ : } {ε : } (hε : 0 < ε) (hδ : 0 δ) (a : E) (b : E) :
Metric.ball a ε + Metric.closedBall b δ = Metric.ball (a + b) (ε + δ)
theorem ball_sub_closedBall {E : Type u_2} [SeminormedAddCommGroup E] [NormedSpace E] {δ : } {ε : } (hε : 0 < ε) (hδ : 0 δ) (a : E) (b : E) :
Metric.ball a ε - Metric.closedBall b δ = Metric.ball (a - b) (ε + δ)
theorem closedBall_add_ball {E : Type u_2} [SeminormedAddCommGroup E] [NormedSpace E] {δ : } {ε : } (hε : 0 ε) (hδ : 0 < δ) (a : E) (b : E) :
Metric.closedBall a ε + Metric.ball b δ = Metric.ball (a + b) (ε + δ)
theorem closedBall_sub_ball {E : Type u_2} [SeminormedAddCommGroup E] [NormedSpace E] {δ : } {ε : } (hε : 0 ε) (hδ : 0 < δ) (a : E) (b : E) :
Metric.closedBall a ε - Metric.ball b δ = Metric.ball (a - b) (ε + δ)
theorem closedBall_add_closedBall {E : Type u_2} [SeminormedAddCommGroup E] [NormedSpace E] {δ : } {ε : } [ProperSpace E] (hε : 0 ε) (hδ : 0 δ) (a : E) (b : E) :
theorem closedBall_sub_closedBall {E : Type u_2} [SeminormedAddCommGroup E] [NormedSpace E] {δ : } {ε : } [ProperSpace E] (hε : 0 ε) (hδ : 0 δ) (a : E) (b : E) :
theorem smul_closedBall {𝕜 : Type u_1} {E : Type u_2} [NormedField 𝕜] [NormedAddCommGroup E] [NormedSpace 𝕜 E] (c : 𝕜) (x : E) {r : } (hr : 0 r) :
theorem smul_closedUnitBall {𝕜 : Type u_1} {E : Type u_2} [NormedField 𝕜] [NormedAddCommGroup E] [NormedSpace 𝕜 E] (c : 𝕜) :

In a real normed space, the image of the unit closed ball under multiplication by a nonnegative number r is the closed ball of radius r with center at the origin.

@[simp]

In a nontrivial real normed space, a sphere is nonempty if and only if its radius is nonnegative.

theorem smul_sphere {𝕜 : Type u_1} {E : Type u_2} [NormedField 𝕜] [NormedAddCommGroup E] [NormedSpace 𝕜 E] [NormedSpace E] [Nontrivial E] (c : 𝕜) (x : E) {r : } (hr : 0 r) :
theorem affinity_unitBall {E : Type u_2} [NormedAddCommGroup E] [NormedSpace E] {r : } (hr : 0 < r) (x : E) :

Any ball Metric.ball x r, 0 < r is the image of the unit ball under fun y ↦ x + r • y.

theorem affinity_unitClosedBall {E : Type u_2} [NormedAddCommGroup E] [NormedSpace E] {r : } (hr : 0 r) (x : E) :

Any closed ball Metric.closedBall x r, 0 ≤ r is the image of the unit closed ball under fun y ↦ x + r • y.