mathlib documentation

analysis.normed_space.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 smul_ball {π•œ : Type u_1} [normed_field π•œ] {E : Type u_2} [semi_normed_group E] [normed_space π•œ E] {c : π•œ} (hc : c β‰  0) (x : E) (r : ℝ) :
theorem smul_sphere' {π•œ : Type u_1} [normed_field π•œ] {E : Type u_2} [semi_normed_group E] [normed_space π•œ E] {c : π•œ} (hc : c β‰  0) (x : E) (r : ℝ) :
@[simp]
theorem normed_space.sphere_nonempty {E : Type u_1} [normed_group E] [normed_space ℝ E] [nontrivial E] {x : E} {r : ℝ} :

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

theorem smul_sphere {π•œ : Type u_1} [normed_field π•œ] {E : Type u_2} [normed_group E] [normed_space π•œ E] [normed_space ℝ E] [nontrivial E] (c : π•œ) (x : E) {r : ℝ} (hr : 0 ≀ r) :
theorem smul_closed_ball' {π•œ : Type u_1} [normed_field π•œ] {E : Type u_2} [semi_normed_group E] [normed_space π•œ E] {c : π•œ} (hc : c β‰  0) (x : E) (r : ℝ) :
theorem metric.bounded.smul {π•œ : Type u_1} [normed_field π•œ] {E : Type u_2} [semi_normed_group E] [normed_space π•œ E] {s : set E} (hs : metric.bounded s) (c : π•œ) :
theorem eventually_singleton_add_smul_subset {π•œ : Type u_1} [normed_field π•œ] {E : Type u_2} [semi_normed_group E] [normed_space π•œ E] {x : E} {s : set E} (hs : metric.bounded s) {u : set E} (hu : u ∈ 𝓝 x) :
βˆ€αΆ  (r : π•œ) in 𝓝 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 set_smul_mem_nhds_zero {π•œ : Type u_1} [normed_field π•œ] {E : Type u_2} [semi_normed_group E] [normed_space π•œ E] {s : set E} (hs : s ∈ 𝓝 0) {c : π•œ} (hc : c β‰  0) :
theorem set_smul_mem_nhds_zero_iff {π•œ : Type u_1} [normed_field π•œ] {E : Type u_2} [semi_normed_group E] [normed_space π•œ E] (s : set E) {c : π•œ} (hc : c β‰  0) :
theorem smul_closed_ball {π•œ : Type u_1} [normed_field π•œ] {E : Type u_2} [normed_group E] [normed_space π•œ E] (c : π•œ) (x : E) {r : ℝ} (hr : 0 ≀ r) :