Continuous functions on a compact space #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
Continuous functions C(α, β)
from a compact space α
to a metric space β
are automatically bounded, and so acquire various structures inherited from α →ᵇ β
.
This file transfers these structures, and restates some lemmas characterising these structures.
If you need a lemma which is proved about α →ᵇ β
but not for C(α, β)
when α
is compact,
you should restate it here. You can also use
bounded_continuous_function.equiv_continuous_map_of_compact
to move functions back and forth.
When α
is compact, the bounded continuous maps α →ᵇ β
are
equivalent to C(α, β)
.
Equations
When α
is compact, the bounded continuous maps α →ᵇ 𝕜
are
additively equivalent to C(α, 𝕜)
.
Equations
- continuous_map.add_equiv_bounded_of_compact α β = {to_fun := (bounded_continuous_function.to_continuous_map_add_hom α β).to_fun, inv_fun := (continuous_map.equiv_bounded_of_compact α β).symm.inv_fun, left_inv := _, right_inv := _, map_add' := _}.symm
When α
is compact, and β
is a metric space, the bounded continuous maps α →ᵇ β
are
isometric to C(α, β)
.
Equations
- continuous_map.isometry_equiv_bounded_of_compact α β = {to_equiv := continuous_map.equiv_bounded_of_compact α β _inst_3, isometry_to_fun := _}
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
See also continuous_map.continuous_eval'
See also continuous_map.continuous_eval_const
See also continuous_map.continuous_coe'
Equations
- continuous_map.has_norm = {norm := λ (x : C(α, E)), has_dist.dist x 0}
Equations
- continuous_map.normed_add_comm_group = {to_has_norm := {norm := has_norm.norm continuous_map.has_norm}, to_add_comm_group := {add := add_comm_group.add continuous_map.add_comm_group, add_assoc := _, zero := add_comm_group.zero continuous_map.add_comm_group, zero_add := _, add_zero := _, nsmul := add_comm_group.nsmul continuous_map.add_comm_group, nsmul_zero' := _, nsmul_succ' := _, neg := add_comm_group.neg continuous_map.add_comm_group, sub := add_comm_group.sub continuous_map.add_comm_group, sub_eq_add_neg := _, zsmul := add_comm_group.zsmul continuous_map.add_comm_group, zsmul_zero' := _, zsmul_succ' := _, zsmul_neg' := _, add_left_neg := _, add_comm := _}, to_metric_space := {to_pseudo_metric_space := {to_has_dist := {dist := has_dist.dist pseudo_metric_space.to_has_dist}, dist_self := _, dist_comm := _, dist_triangle := _, edist := pseudo_metric_space.edist metric_space.to_pseudo_metric_space, edist_dist := _, to_uniform_space := pseudo_metric_space.to_uniform_space metric_space.to_pseudo_metric_space, uniformity_dist := _, to_bornology := pseudo_metric_space.to_bornology metric_space.to_pseudo_metric_space, cobounded_sets := _}, eq_of_dist_eq_zero := _}, dist_eq := _}
Distance between the images of any two points is at most twice the norm of the function.
Equations
- continuous_map.normed_ring = {to_has_norm := normed_add_comm_group.to_has_norm infer_instance, to_ring := {add := add_comm_group.add normed_add_comm_group.to_add_comm_group, add_assoc := _, zero := add_comm_group.zero normed_add_comm_group.to_add_comm_group, zero_add := _, add_zero := _, nsmul := add_comm_group.nsmul normed_add_comm_group.to_add_comm_group, nsmul_zero' := _, nsmul_succ' := _, neg := add_comm_group.neg normed_add_comm_group.to_add_comm_group, sub := add_comm_group.sub normed_add_comm_group.to_add_comm_group, sub_eq_add_neg := _, zsmul := add_comm_group.zsmul normed_add_comm_group.to_add_comm_group, zsmul_zero' := _, zsmul_succ' := _, zsmul_neg' := _, add_left_neg := _, add_comm := _, int_cast := ring.int_cast continuous_map.ring, nat_cast := ring.nat_cast continuous_map.ring, one := ring.one continuous_map.ring, nat_cast_zero := _, nat_cast_succ := _, int_cast_of_nat := _, int_cast_neg_succ_of_nat := _, mul := ring.mul continuous_map.ring, mul_assoc := _, one_mul := _, mul_one := _, npow := ring.npow continuous_map.ring, npow_zero' := _, npow_succ' := _, left_distrib := _, right_distrib := _}, to_metric_space := normed_add_comm_group.to_metric_space infer_instance, dist_eq := _, norm_mul := _}
Equations
- continuous_map.normed_space = {to_module := continuous_map.module continuous_map.normed_space._proof_2, norm_smul_le := _}
When α
is compact and 𝕜
is a normed field,
the 𝕜
-algebra of bounded continuous maps α →ᵇ β
is
𝕜
-linearly isometric to C(α, β)
.
Equations
- continuous_map.linear_isometry_bounded_of_compact α E 𝕜 = {to_linear_equiv := {to_fun := (continuous_map.add_equiv_bounded_of_compact α E).to_fun, map_add' := _, map_smul' := _, inv_fun := (continuous_map.add_equiv_bounded_of_compact α E).inv_fun, left_inv := _, right_inv := _}, norm_map' := _}
The evaluation at a point, as a continuous linear map from C(α, 𝕜)
to 𝕜
.
Equations
- continuous_map.normed_algebra = {to_algebra := continuous_map.algebra continuous_map.normed_algebra._proof_1, norm_smul_le := _}
We now set up some declarations making it convenient to use uniform continuity.
An arbitrarily chosen modulus of uniform continuity for a given function f
and ε > 0
.
Equations
- f.modulus ε h = classical.some _
Postcomposition of continuous functions into a normed module by a continuous linear map is a
continuous linear map.
Transferred version of continuous_linear_map.comp_left_continuous_bounded
,
upgraded version of continuous_linear_map.comp_left_continuous
,
similar to linear_map.comp_left
.
Equations
- continuous_linear_map.comp_left_continuous_compact X g = (continuous_map.linear_isometry_bounded_of_compact X γ 𝕜).symm.to_linear_isometry.to_continuous_linear_map.comp ((continuous_linear_map.comp_left_continuous_bounded X g).comp (continuous_map.linear_isometry_bounded_of_compact X β 𝕜).to_linear_isometry.to_continuous_linear_map)
We now setup variations on comp_right_* f
, where f : C(X, Y)
(that is, precomposition by a continuous map),
as a morphism C(Y, T) → C(X, T)
, respecting various types of structure.
In particular:
comp_right_continuous_map
, the bundled continuous map (for this we needX Y
compact).comp_right_homeomorph
, when we precompose by a homeomorphism.comp_right_alg_hom
, whenT = R
is a topological ring.
Precomposition by a continuous map is itself a continuous map between spaces of continuous maps.
Equations
- continuous_map.comp_right_continuous_map T f = {to_fun := λ (g : C(Y, T)), g.comp f, continuous_to_fun := _}
Precomposition by a homeomorphism is itself a homeomorphism between spaces of continuous maps.
Equations
- continuous_map.comp_right_homeomorph T f = {to_equiv := {to_fun := ⇑(continuous_map.comp_right_continuous_map T f.to_continuous_map), inv_fun := ⇑(continuous_map.comp_right_continuous_map T f.symm.to_continuous_map), left_inv := _, right_inv := _}, continuous_to_fun := _, continuous_inv_fun := _}
Local normal convergence #
A sum of continuous functions (on a locally compact space) is "locally normally convergent" if the
sum of its sup-norms on any compact subset is summable. This implies convergence in the topology
of C(X, E)
(i.e. locally uniform convergence).
Star structures #
In this section, if β
is a normed ⋆-group, then so is the space of
continuous functions from α
to β
, by using the star operation pointwise.
Furthermore, if α
is compact and β
is a C⋆-ring, then C(α, β)
is a C⋆-ring.