mathlib3 documentation

analysis.normed_space.pointwise

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

THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.

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} [seminormed_add_comm_group 𝕜] [seminormed_add_comm_group E] [smul_zero_class 𝕜 E] [has_bounded_smul 𝕜 E] (c : 𝕜) (s : set E) :
theorem ediam_smul₀ {𝕜 : Type u_1} {E : Type u_2} [normed_division_ring 𝕜] [seminormed_add_comm_group E] [module 𝕜 E] [has_bounded_smul 𝕜 E] (c : 𝕜) (s : set E) :
theorem diam_smul₀ {𝕜 : Type u_1} {E : Type u_2} [normed_division_ring 𝕜] [seminormed_add_comm_group E] [module 𝕜 E] [has_bounded_smul 𝕜 E] (c : 𝕜) (x : set E) :
theorem inf_edist_smul₀ {𝕜 : Type u_1} {E : Type u_2} [normed_division_ring 𝕜] [seminormed_add_comm_group E] [module 𝕜 E] [has_bounded_smul 𝕜 E] {c : 𝕜} (hc : c 0) (s : set E) (x : E) :
theorem inf_dist_smul₀ {𝕜 : Type u_1} {E : Type u_2} [normed_division_ring 𝕜] [seminormed_add_comm_group E] [module 𝕜 E] [has_bounded_smul 𝕜 E] {c : 𝕜} (hc : c 0) (s : set E) (x : E) :
theorem smul_ball {𝕜 : Type u_1} {E : Type u_2} [normed_field 𝕜] [seminormed_add_comm_group E] [normed_space 𝕜 E] {c : 𝕜} (hc : c 0) (x : E) (r : ) :
theorem smul_unit_ball {𝕜 : Type u_1} {E : Type u_2} [normed_field 𝕜] [seminormed_add_comm_group E] [normed_space 𝕜 E] {c : 𝕜} (hc : c 0) :
theorem smul_sphere' {𝕜 : Type u_1} {E : Type u_2} [normed_field 𝕜] [seminormed_add_comm_group E] [normed_space 𝕜 E] {c : 𝕜} (hc : c 0) (x : E) (r : ) :
theorem smul_closed_ball' {𝕜 : Type u_1} {E : Type u_2} [normed_field 𝕜] [seminormed_add_comm_group E] [normed_space 𝕜 E] {c : 𝕜} (hc : c 0) (x : E) (r : ) :
theorem metric.bounded.smul {𝕜 : Type u_1} {E : Type u_2} [normed_field 𝕜] [seminormed_add_comm_group E] [normed_space 𝕜 E] {s : set E} (hs : metric.bounded s) (c : 𝕜) :
theorem eventually_singleton_add_smul_subset {𝕜 : Type u_1} {E : Type u_2} [normed_field 𝕜] [seminormed_add_comm_group E] [normed_space 𝕜 E] {x : E} {s : set E} (hs : metric.bounded 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_unit_ball_of_pos {E : Type u_2} [seminormed_add_comm_group E] [normed_space 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 exists_dist_eq {E : Type u_2} [seminormed_add_comm_group E] [normed_space E] (x z : E) {a b : } (ha : 0 a) (hb : 0 b) (hab : a + b = 1) :
theorem exists_dist_le_le {E : Type u_2} [seminormed_add_comm_group E] [normed_space E] {x z : E} {δ ε : } (hδ : 0 δ) (hε : 0 ε) (h : has_dist.dist x z ε + δ) :
(y : E), has_dist.dist x y δ has_dist.dist y z ε
theorem exists_dist_le_lt {E : Type u_2} [seminormed_add_comm_group E] [normed_space E] {x z : E} {δ ε : } (hδ : 0 δ) (hε : 0 < ε) (h : has_dist.dist x z < ε + δ) :
(y : E), has_dist.dist x y δ has_dist.dist y z < ε
theorem exists_dist_lt_le {E : Type u_2} [seminormed_add_comm_group E] [normed_space E] {x z : E} {δ ε : } (hδ : 0 < δ) (hε : 0 ε) (h : has_dist.dist x z < ε + δ) :
(y : E), has_dist.dist x y < δ has_dist.dist y z ε
theorem exists_dist_lt_lt {E : Type u_2} [seminormed_add_comm_group E] [normed_space E] {x z : E} {δ ε : } (hδ : 0 < δ) (hε : 0 < ε) (h : has_dist.dist x z < ε + δ) :
(y : E), has_dist.dist x y < δ has_dist.dist y z < ε
theorem disjoint_ball_ball_iff {E : Type u_2} [seminormed_add_comm_group E] [normed_space E] {x y : E} {δ ε : } (hδ : 0 < δ) (hε : 0 < ε) :
theorem disjoint_ball_closed_ball_iff {E : Type u_2} [seminormed_add_comm_group E] [normed_space E] {x y : E} {δ ε : } (hδ : 0 < δ) (hε : 0 ε) :
theorem disjoint_closed_ball_ball_iff {E : Type u_2} [seminormed_add_comm_group E] [normed_space E] {x y : E} {δ ε : } (hδ : 0 δ) (hε : 0 < ε) :
theorem disjoint_closed_ball_closed_ball_iff {E : Type u_2} [seminormed_add_comm_group E] [normed_space E] {x y : E} {δ ε : } (hδ : 0 δ) (hε : 0 ε) :
@[simp]
theorem inf_edist_thickening {E : Type u_2} [seminormed_add_comm_group E] [normed_space E] {δ : } (hδ : 0 < δ) (s : set E) (x : E) :
@[simp]
theorem thickening_thickening {E : Type u_2} [seminormed_add_comm_group E] [normed_space E] {δ ε : } (hε : 0 < ε) (hδ : 0 < δ) (s : set E) :
@[simp]
theorem cthickening_thickening {E : Type u_2} [seminormed_add_comm_group E] [normed_space E] {δ ε : } (hε : 0 ε) (hδ : 0 < δ) (s : set E) :
@[simp]
theorem closure_thickening {E : Type u_2} [seminormed_add_comm_group E] [normed_space E] {δ : } (hδ : 0 < δ) (s : set E) :
@[simp]
theorem thickening_cthickening {E : Type u_2} [seminormed_add_comm_group E] [normed_space E] {δ ε : } (hε : 0 < ε) (hδ : 0 δ) (s : set E) :
@[simp]
theorem cthickening_cthickening {E : Type u_2} [seminormed_add_comm_group E] [normed_space E] {δ ε : } (hε : 0 ε) (hδ : 0 δ) (s : set E) :
@[simp]
theorem thickening_ball {E : Type u_2} [seminormed_add_comm_group E] [normed_space E] {δ ε : } (hε : 0 < ε) (hδ : 0 < δ) (x : E) :
@[simp]
theorem thickening_closed_ball {E : Type u_2} [seminormed_add_comm_group E] [normed_space E] {δ ε : } (hε : 0 < ε) (hδ : 0 δ) (x : E) :
@[simp]
theorem cthickening_ball {E : Type u_2} [seminormed_add_comm_group E] [normed_space E] {δ ε : } (hε : 0 ε) (hδ : 0 < δ) (x : E) :
@[simp]
theorem cthickening_closed_ball {E : Type u_2} [seminormed_add_comm_group E] [normed_space E] {δ ε : } (hε : 0 ε) (hδ : 0 δ) (x : E) :
theorem ball_add_ball {E : Type u_2} [seminormed_add_comm_group E] [normed_space E] {δ ε : } (hε : 0 < ε) (hδ : 0 < δ) (a b : E) :
metric.ball a ε + metric.ball b δ = metric.ball (a + b) + δ)
theorem ball_sub_ball {E : Type u_2} [seminormed_add_comm_group E] [normed_space E] {δ ε : } (hε : 0 < ε) (hδ : 0 < δ) (a b : E) :
metric.ball a ε - metric.ball b δ = metric.ball (a - b) + δ)
theorem ball_add_closed_ball {E : Type u_2} [seminormed_add_comm_group E] [normed_space E] {δ ε : } (hε : 0 < ε) (hδ : 0 δ) (a b : E) :
metric.ball a ε + metric.closed_ball b δ = metric.ball (a + b) + δ)
theorem ball_sub_closed_ball {E : Type u_2} [seminormed_add_comm_group E] [normed_space E] {δ ε : } (hε : 0 < ε) (hδ : 0 δ) (a b : E) :
metric.ball a ε - metric.closed_ball b δ = metric.ball (a - b) + δ)
theorem closed_ball_add_ball {E : Type u_2} [seminormed_add_comm_group E] [normed_space E] {δ ε : } (hε : 0 ε) (hδ : 0 < δ) (a b : E) :
metric.closed_ball a ε + metric.ball b δ = metric.ball (a + b) + δ)
theorem closed_ball_sub_ball {E : Type u_2} [seminormed_add_comm_group E] [normed_space E] {δ ε : } (hε : 0 ε) (hδ : 0 < δ) (a b : E) :
metric.closed_ball a ε - metric.ball b δ = metric.ball (a - b) + δ)
theorem closed_ball_add_closed_ball {E : Type u_2} [seminormed_add_comm_group E] [normed_space E] {δ ε : } [proper_space E] (hε : 0 ε) (hδ : 0 δ) (a b : E) :
theorem closed_ball_sub_closed_ball {E : Type u_2} [seminormed_add_comm_group E] [normed_space E] {δ ε : } [proper_space E] (hε : 0 ε) (hδ : 0 δ) (a b : E) :
theorem smul_closed_ball {𝕜 : Type u_1} {E : Type u_2} [normed_field 𝕜] [normed_add_comm_group E] [normed_space 𝕜 E] (c : 𝕜) (x : E) {r : } (hr : 0 r) :
theorem smul_closed_unit_ball {𝕜 : Type u_1} {E : Type u_2} [normed_field 𝕜] [normed_add_comm_group E] [normed_space 𝕜 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} [normed_field 𝕜] [normed_add_comm_group E] [normed_space 𝕜 E] [normed_space E] [nontrivial E] (c : 𝕜) (x : E) {r : } (hr : 0 r) :
theorem affinity_unit_ball {E : Type u_2} [normed_add_comm_group E] [normed_space E] {r : } (hr : 0 < r) (x : E) :

Any ball metric.ball x r, 0 < r is the image of the unit ball under λ y, x + r • y.

theorem affinity_unit_closed_ball {E : Type u_2} [normed_add_comm_group E] [normed_space E] {r : } (hr : 0 r) (x : E) :

Any closed ball metric.closed_ball x r, 0 ≤ r is the image of the unit closed ball under λ y, x + r • y.