Continuous functions vanishing at infinity #
The type of continuous functions vanishing at infinity. When the domain is compact
C(α, β) ≃ C₀(α, β)
via the identity map. When the codomain is a metric space, every continuous
map which vanishes at infinity is a bounded continuous function. When the domain is a locally
compact space, this type has nice properties.
TODO #
- Create more intances of algebraic structures (e.g.,
NonUnitalSemiring
) once the necessary type classes (e.g.,TopologicalRing
) are sufficiently generalized. - Relate the unitization of
C₀(α, β)
to the Alexandroff compactification.
- toFun : α → β
- continuous_toFun : Continuous s.toFun
- zero_at_infty' : Filter.Tendsto s.toFun (Filter.cocompact α) (nhds 0)
The function tends to zero along the
cocompact
filter.
C₀(α, β)
is the type of continuous functions α → β
which vanish at infinity from a
topological space to a metric space with a zero element.
When possible, instead of parametrizing results over (f : C₀(α, β))
,
you should parametrize over (F : Type*) [ZeroAtInftyContinuousMapClass F α β] (f : F)
.
When you extend this structure, make sure to extend ZeroAtInftyContinuousMapClass
.
Instances For
C₀(α, β)
is the type of continuous functions α → β
which vanish at infinity from a
topological space to a metric space with a zero element.
When possible, instead of parametrizing results over (f : C₀(α, β))
,
you should parametrize over (F : Type*) [ZeroAtInftyContinuousMapClass F α β] (f : F)
.
When you extend this structure, make sure to extend ZeroAtInftyContinuousMapClass
.
Instances For
C₀(α, β)
is the type of continuous functions α → β
which vanish at infinity from a
topological space to a metric space with a zero element.
When possible, instead of parametrizing results over (f : C₀(α, β))
,
you should parametrize over (F : Type*) [ZeroAtInftyContinuousMapClass F α β] (f : F)
.
When you extend this structure, make sure to extend ZeroAtInftyContinuousMapClass
.
Instances For
- coe : F → α → β
- coe_injective' : Function.Injective FunLike.coe
- map_continuous : ∀ (f : F), Continuous ↑f
- zero_at_infty : ∀ (f : F), Filter.Tendsto (↑f) (Filter.cocompact α) (nhds 0)
Each member of the class tends to zero along the
cocompact
filter.
ZeroAtInftyContinuousMapClass F α β
states that F
is a type of continuous maps which
vanish at infinity.
You should also extend this typeclass when you extend ZeroAtInftyContinuousMap
.
Instances
Helper instance for when there's too many metavariables to apply FunLike.hasCoeToFun
directly.
Copy of a ZeroAtInftyContinuousMap
with a new toFun
equal to the old one. Useful
to fix definitional equalities.
Instances For
A continuous function on a compact space is automatically a continuous function vanishing at infinity.
Instances For
A continuous function on a compact space is automatically a continuous function vanishing at infinity. This is not an instance to avoid type class loops.
Instances For
Algebraic structure #
Whenever β
has suitable algebraic structure and a compatible topological structure, then
C₀(α, β)
inherits a corresponding algebraic structure. The primary exception to this is that
C₀(α, β)
will not have a multiplicative identity.
Metric structure #
When β
is a metric space, then every element of C₀(α, β)
is bounded, and so there is a natural
inclusion map ZeroAtInftyContinuousMap.toBcf : C₀(α, β) → (α →ᵇ β)
. Via this map C₀(α, β)
inherits a metric as the pullback of the metric on α →ᵇ β
. Moreover, this map has closed range
in α →ᵇ β
and consequently C₀(α, β)
is a complete space whenever β
is complete.
Construct a bounded continuous function from a continuous function vanishing at infinity.
Instances For
The type of continuous functions vanishing at infinity, with the uniform distance induced by the
inclusion ZeroAtInftyContinuousMap.toBcf
, is a metric space.
Convergence in the metric on C₀(α, β)
is uniform convergence.
Continuous functions vanishing at infinity taking values in a complete space form a complete space.
Normed space #
The norm structure on C₀(α, β)
is the one induced by the inclusion toBcf : C₀(α, β) → (α →ᵇ b)
,
viewed as an additive monoid homomorphism. Then C₀(α, β)
is naturally a normed space over a normed
field 𝕜
whenever β
is as well.
Star structure #
It is possible to equip C₀(α, β)
with a pointwise star
operation whenever there is a continuous
star : β → β
for which star (0 : β) = 0
. We don't have quite this weak a typeclass, but
StarAddMonoid
is close enough.
The StarAddMonoid
and NormedStarGroup
classes on C₀(α, β)
are inherited from their
counterparts on α →ᵇ β
. Ultimately, when β
is a C⋆-ring, then so is C₀(α, β)
.
C₀ as a functor #
For each β
with sufficient structure, there is a contravariant functor C₀(-, β)
from the
category of topological spaces with morphisms given by CocompactMap
s.
Composition of a continuous function vanishing at infinity with a cocompact map yields another continuous function vanishing at infinity.
Instances For
Composition as an additive monoid homomorphism.
Instances For
Composition as a semigroup homomorphism.
Instances For
Composition as a linear map.
Instances For
Composition as a non-unital algebra homomorphism.