Continuous bundled maps #
In this file we define the type ContinuousMap
of continuous bundled maps.
We use the FunLike
design, so each type of morphisms has a companion typeclass which is meant to
be satisfied by itself and all stricter types.
- toFun : α → β
The function
α → β
- continuous_toFun : Continuous s.toFun
Proposition that
toFun
is continuous
The type of continuous maps from α
to β
.
When possible, instead of parametrizing results over (f : C(α, β))
,
you should parametrize over {F : Type*} [ContinuousMapClass F α β] (f : F)
.
When you extend this structure, make sure to extend ContinuousMapClass
.
Instances For
- coe : F → α → β
- coe_injective' : Function.Injective FunLike.coe
- map_continuous : ∀ (f : F), Continuous ↑f
Continuity
ContinuousMapClass F α β
states that F
is a type of continuous maps.
You should extend this class when you extend ContinuousMap
.
Instances
Coerce a bundled morphism with a ContinuousMapClass
instance to a ContinuousMap
.
Instances For
Continuous maps #
See note [custom simps projection].
Instances For
Copy of a ContinuousMap
with a new toFun
equal to the old one. Useful to fix definitional
equalities.
Instances For
Deprecated. Use map_continuous
instead.
Deprecated. Use map_continuousAt
instead.
Deprecated. Use FunLike.congr_fun
instead.
Deprecated. Use FunLike.congr_arg
instead.
The continuous functions from α
to β
are the same as the plain functions when α
is discrete.
Instances For
The identity as a continuous map.
Instances For
The constant map as a continuous map.
Instances For
Function.const α b
as a bundled continuous function of b
.
Instances For
The composition of continuous maps, as a continuous map.
Instances For
Prod.fst : (x, y) ↦ x
as a bundled continuous map.
Instances For
Prod.snd : (x, y) ↦ y
as a bundled continuous map.
Instances For
Given two continuous maps f
and g
, this is the continuous map x ↦ (f x, g x)
.
Instances For
Given two continuous maps f
and g
, this is the continuous map (x, y) ↦ (f x, g y)
.
Instances For
Prod.swap
bundled as a ContinuousMap
.
Instances For
Sigma.mk i
as a bundled continuous map.
Instances For
Abbreviation for product of continuous maps, which is continuous
Instances For
Evaluation at point as a bundled continuous map.
Instances For
Combine a collection of bundled continuous maps C(X i, Y i)
into a bundled continuous map
C(∀ i, X i, ∀ i, Y i)
.
Instances For
The restriction of a continuous function α → β
to a subset s
of α
.
Instances For
The restriction of a continuous map to the preimage of a set.
Instances For
A family φ i
of continuous maps C(S i, β)
, where the domains S i
contain a neighbourhood
of each point in α
and the functions φ i
agree pairwise on intersections, can be glued to
construct a continuous map in C(α, β)
.
Instances For
A family F s
of continuous maps C(s, β)
, where (1) the domains s
are taken from a set A
of sets in α
which contain a neighbourhood of each point in α
and (2) the functions F s
agree
pairwise on intersections, can be glued to construct a continuous map in C(α, β)
.
Instances For
The forward direction of a homeomorphism, as a bundled continuous map.
Instances For
Homeomorph.toContinuousMap
as a coercion.
Left inverse to a continuous map from a homeomorphism, mirroring Equiv.symm_comp_self
.
Right inverse to a continuous map from a homeomorphism, mirroring Equiv.self_comp_symm
.