Cocompact continuous maps #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
The type of cocompact continuous maps are those which tend to the cocompact filter on the codomain along the cocompact filter on the domain. When the domain and codomain are Hausdorff, this is equivalent to many other conditions, including that preimages of compact sets are compact.
Cocompact continuous maps #
- to_continuous_map : C(α, β)
- cocompact_tendsto' : filter.tendsto self.to_continuous_map.to_fun (filter.cocompact α) (filter.cocompact β)
A cocompact continuous map is a continuous function between topological spaces which
tends to the cocompact filter along the cocompact filter. Functions for which preimages of compact
sets are compact always satisfy this property, and the converse holds for cocompact continuous maps
when the codomain is Hausdorff (see cocompact_map.tendsto_of_forall_preimage
and
cocompact_map.is_compact_preimage
).
Cocompact maps thus generalise proper maps, with which they correspond when the codomain is Hausdorff.
Instances for cocompact_map
- cocompact_map.has_sizeof_inst
- cocompact_map_class.cocompact_map.has_coe_t
- cocompact_map.cocompact_map_class
- cocompact_map.has_coe_to_fun
- cocompact_map.inhabited
- coe : F → Π (a : α), (λ (_x : α), β) a
- coe_injective' : function.injective cocompact_map_class.coe
- map_continuous : ∀ (f : F), continuous ⇑f
- cocompact_tendsto : ∀ (f : F), filter.tendsto ⇑f (filter.cocompact α) (filter.cocompact β)
cocompact_map_class F α β
states that F
is a type of cocompact continuous maps.
You should also extend this typeclass when you extend cocompact_map
.
Instances of this typeclass
Instances of other typeclasses for cocompact_map_class
- cocompact_map_class.has_sizeof_inst
Equations
- cocompact_map_class.cocompact_map.has_coe_t = {coe := λ (f : F), {to_continuous_map := ↑f, cocompact_tendsto' := _}}
Equations
- cocompact_map.cocompact_map_class = {coe := λ (f : cocompact_map α β), f.to_continuous_map.to_fun, coe_injective' := _, map_continuous := _, cocompact_tendsto := _}
Helper instance for when there's too many metavariables to apply fun_like.has_coe_to_fun
directly.
Copy of a cocompact_map
with a new to_fun
equal to the old one. Useful
to fix definitional equalities.
Equations
- f.copy f' h = {to_continuous_map := {to_fun := f', continuous_to_fun := _}, cocompact_tendsto' := _}
The identity as a cocompact continuous map.
Equations
- cocompact_map.id α = {to_continuous_map := continuous_map.id α _inst_1, cocompact_tendsto' := _}
Equations
- cocompact_map.inhabited = {default := cocompact_map.id α _inst_1}
The composition of cocompact continuous maps, as a cocompact continuous map.
Equations
- f.comp g = {to_continuous_map := f.to_continuous_map.comp ↑g, cocompact_tendsto' := _}
If the codomain is Hausdorff, preimages of compact sets are compact under a cocompact continuous map.
A homemomorphism is a cocompact map.
Equations
- f.to_cocompact_map = {to_continuous_map := {to_fun := ⇑f, continuous_to_fun := _}, cocompact_tendsto' := _}