Bounded continuous functions
The type of bounded continuous functions taking values in a metric space, with the uniform distance.
The type of bounded continuous functions from a topological space to a metric space
Equations
- bounded_continuous_function α β = {f // continuous f ∧ ∃ (C : ℝ), ∀ (x y : α), has_dist.dist (f x) (f y) ≤ C}
Equations
- bounded_continuous_function.has_coe_to_fun = {F := λ (x : bounded_continuous_function α β), α → β, coe := subtype.val (λ (f : α → β), continuous f ∧ ∃ (C : ℝ), ∀ (x y : α), has_dist.dist (f x) (f y) ≤ C)}
If a function is continuous on a compact space, it is automatically bounded, and therefore gives rise to an element of the type of bounded continuous functions
Equations
- bounded_continuous_function.mk_of_compact f hf = ⟨f, _⟩
If a function is bounded on a discrete space, it is automatically continuous, and therefore gives rise to an element of the type of bounded continuous functions
Equations
- bounded_continuous_function.mk_of_discrete f hf = ⟨f, _⟩
The uniform distance between two bounded continuous functions
Equations
- bounded_continuous_function.has_dist = {dist := λ (f g : bounded_continuous_function α β), has_Inf.Inf {C : ℝ | 0 ≤ C ∧ ∀ (x : α), has_dist.dist (⇑f x) (⇑g x) ≤ C}}
The pointwise distance is controlled by the distance between functions, by definition
The distance between two functions is controlled by the supremum of the pointwise distances
On an empty space, bounded continuous functions are at distance 0
The type of bounded continuous functions, with the uniform distance, is a metric space.
Equations
- bounded_continuous_function.metric_space = {to_has_dist := bounded_continuous_function.has_dist _inst_2, dist_self := _, eq_of_dist_eq_zero := _, dist_comm := _, dist_triangle := _, edist := λ (x y : bounded_continuous_function α β), ennreal.of_real ((λ (f g : bounded_continuous_function α β), has_Inf.Inf {C : ℝ | 0 ≤ C ∧ ∀ (x : α), has_dist.dist (⇑f x) (⇑g x) ≤ C}) x y), edist_dist := _, to_uniform_space := uniform_space_of_dist (λ (f g : bounded_continuous_function α β), has_Inf.Inf {C : ℝ | 0 ≤ C ∧ ∀ (x : α), has_dist.dist (⇑f x) (⇑g x) ≤ C}) bounded_continuous_function.metric_space._proof_6 bounded_continuous_function.metric_space._proof_7 bounded_continuous_function.metric_space._proof_8, uniformity_dist := _}
Constant as a continuous bounded function.
Equations
- bounded_continuous_function.const α b = ⟨λ (x : α), b, _⟩
If the target space is inhabited, so is the space of bounded continuous functions
Equations
The evaluation map is continuous, as a joint function of u
and x
In particular, when x
is fixed, f → f x
is continuous
When f
is fixed, x → f x
is also continuous, by definition
Bounded continuous functions taking values in a complete space form a complete space.
Equations
Composition (in the target) of a bounded continuous function with a Lipschitz map again gives a bounded continuous function
Equations
- bounded_continuous_function.comp G H f = ⟨λ (x : α), G (⇑f x), _⟩
The composition operator (in the target) with a Lipschitz map is Lipschitz
The composition operator (in the target) with a Lipschitz map is uniformly continuous
The composition operator (in the target) with a Lipschitz map is continuous
Restriction (in the target) of a bounded continuous function taking values in a subset
Equations
- bounded_continuous_function.cod_restrict s f H = ⟨set.cod_restrict ⇑f s H, _⟩
First version, with pointwise equicontinuity and range in a compact space
Second version, with pointwise equicontinuity and range in a compact subset
Third (main) version, with pointwise equicontinuity and range in a compact subset, but without closedness. The closure is then compact
Equations
Equations
- bounded_continuous_function.has_norm = {norm := λ (u : bounded_continuous_function α β), has_dist.dist u 0}
The norm of a bounded continuous function is the supremum of ∥f x∥
.
We use Inf
to ensure that the definition works if α
has no elements.
Distance between the images of any two points is at most twice the norm of the function.
The norm of a function is controlled by the supremum of the pointwise norms
Norm of const α b
is less than or equal to ∥b∥
. If α
is nonempty,
then it is equal to ∥b∥
.
Constructing a bounded continuous function from a uniformly bounded continuous function taking values in a normed group.
Equations
- bounded_continuous_function.of_normed_group f Hf C H = ⟨λ (n : α), f n, _⟩
Constructing a bounded continuous function from a uniformly bounded function on a discrete space, taking values in a normed group
Equations
The pointwise sum of two bounded continuous functions is again bounded continuous.
Equations
- bounded_continuous_function.has_add = {add := λ (f g : bounded_continuous_function α β), bounded_continuous_function.of_normed_group (⇑f + ⇑g) _ (∥f∥ + ∥g∥) _}
The pointwise opposite of a bounded continuous function is again bounded continuous.
Equations
- bounded_continuous_function.has_neg = {neg := λ (f : bounded_continuous_function α β), bounded_continuous_function.of_normed_group (-⇑f) _ ∥f∥ _}
Equations
- bounded_continuous_function.add_comm_group = {add := has_add.add bounded_continuous_function.has_add, add_assoc := _, zero := 0, zero_add := _, add_zero := _, neg := has_neg.neg bounded_continuous_function.has_neg, add_left_neg := _, add_comm := _}
Normed space structure
In this section, if β
is a normed space, then we show that the space of bounded
continuous functions from α
to β
inherits a normed space structure, by using
pointwise operations and checking that they are compatible with the uniform distance.
Equations
- bounded_continuous_function.has_scalar = {smul := λ (c : 𝕜) (f : bounded_continuous_function α β), bounded_continuous_function.of_normed_group (c • ⇑f) _ (∥c∥ * ∥f∥) _}
Equations
- bounded_continuous_function.semimodule = semimodule.of_core {to_has_scalar := {smul := has_scalar.smul bounded_continuous_function.has_scalar}, smul_add := _, add_smul := _, mul_smul := _, one_smul := _}
Equations
Normed ring structure
In this section, if R
is a normed ring, then we show that the space of bounded
continuous functions from α
to R
inherits a normed ring structure, by using
pointwise operations and checking that they are compatible with the uniform distance.
Equations
- bounded_continuous_function.ring = {add := add_comm_group.add bounded_continuous_function.add_comm_group, add_assoc := _, zero := add_comm_group.zero bounded_continuous_function.add_comm_group, zero_add := _, add_zero := _, neg := add_comm_group.neg bounded_continuous_function.add_comm_group, add_left_neg := _, add_comm := _, mul := λ (f g : bounded_continuous_function α R), bounded_continuous_function.of_normed_group (⇑f * ⇑g) _ (∥f∥ * ∥g∥) _, mul_assoc := _, one := bounded_continuous_function.const α 1, one_mul := _, mul_one := _, left_distrib := _, right_distrib := _}
Equations
Normed algebra structure
In this section, if γ
is a normed algebra, then we show that the space of bounded
continuous functions from α
to γ
inherits a normed algebra structure, by using
pointwise operations and checking that they are compatible with the uniform distance.
bounded_continuous_function.const
as a ring_hom
.
Equations
- bounded_continuous_function.C = {to_fun := λ (c : 𝕜), bounded_continuous_function.const α (⇑(algebra_map 𝕜 γ) c), map_one' := _, map_mul' := _, map_zero' := _, map_add' := _}
Equations
Structure as normed module over scalar functions
If β
is a normed 𝕜
-space, then we show that the space of bounded continuous
functions from α
to β
is naturally a module over the algebra of bounded continuous
functions from α
to 𝕜
.
Equations
- bounded_continuous_function.has_scalar' = {smul := λ (f : bounded_continuous_function α 𝕜) (g : bounded_continuous_function α β), bounded_continuous_function.of_normed_group (λ (x : α), ⇑f x • ⇑g x) _ (∥f∥ * ∥g∥) _}
Equations
- bounded_continuous_function.module' = semimodule.of_core {to_has_scalar := {smul := has_scalar.smul bounded_continuous_function.has_scalar'}, smul_add := _, add_smul := _, mul_smul := _, one_smul := _}