mathlib3 documentation

topology.continuous_function.cocompact_map

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 #

structure cocompact_map (α : Type u) (β : Type v) [topological_space α] [topological_space β] :
Type (max u v)

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
@[class]
structure cocompact_map_class (F : Type u_1) (α : out_param (Type u_2)) (β : out_param (Type u_3)) [topological_space α] [topological_space β] :
Type (max u_1 u_2 u_3)

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
@[instance]
@[protected, instance]
def cocompact_map.has_coe_to_fun {α : Type u_1} {β : Type u_2} [topological_space α] [topological_space β] :
has_coe_to_fun (cocompact_map α β) (λ (_x : cocompact_map α β), α β)

Helper instance for when there's too many metavariables to apply fun_like.has_coe_to_fun directly.

Equations
@[ext]
theorem cocompact_map.ext {α : Type u_1} {β : Type u_2} [topological_space α] [topological_space β] {f g : cocompact_map α β} (h : (x : α), f x = g x) :
f = g
@[protected]
def cocompact_map.copy {α : Type u_1} {β : Type u_2} [topological_space α] [topological_space β] (f : cocompact_map α β) (f' : α β) (h : f' = f) :

Copy of a cocompact_map with a new to_fun equal to the old one. Useful to fix definitional equalities.

Equations
@[simp]
theorem cocompact_map.coe_copy {α : Type u_1} {β : Type u_2} [topological_space α] [topological_space β] (f : cocompact_map α β) (f' : α β) (h : f' = f) :
(f.copy f' h) = f'
theorem cocompact_map.copy_eq {α : Type u_1} {β : Type u_2} [topological_space α] [topological_space β] (f : cocompact_map α β) (f' : α β) (h : f' = f) :
f.copy f' h = f
@[protected]
def cocompact_map.id (α : Type u_1) [topological_space α] :

The identity as a cocompact continuous map.

Equations
@[simp]
@[protected, instance]
Equations
def cocompact_map.comp {α : Type u_1} {β : Type u_2} {γ : Type u_3} [topological_space α] [topological_space β] [topological_space γ] (f : cocompact_map β γ) (g : cocompact_map α β) :

The composition of cocompact continuous maps, as a cocompact continuous map.

Equations
@[simp]
theorem cocompact_map.coe_comp {α : Type u_1} {β : Type u_2} {γ : Type u_3} [topological_space α] [topological_space β] [topological_space γ] (f : cocompact_map β γ) (g : cocompact_map α β) :
(f.comp g) = f g
@[simp]
theorem cocompact_map.comp_apply {α : Type u_1} {β : Type u_2} {γ : Type u_3} [topological_space α] [topological_space β] [topological_space γ] (f : cocompact_map β γ) (g : cocompact_map α β) (a : α) :
(f.comp g) a = f (g a)
@[simp]
theorem cocompact_map.comp_assoc {α : Type u_1} {β : Type u_2} {γ : Type u_3} {δ : Type u_4} [topological_space α] [topological_space β] [topological_space γ] [topological_space δ] (f : cocompact_map γ δ) (g : cocompact_map β γ) (h : cocompact_map α β) :
(f.comp g).comp h = f.comp (g.comp h)
@[simp]
theorem cocompact_map.id_comp {α : Type u_1} {β : Type u_2} [topological_space α] [topological_space β] (f : cocompact_map α β) :
@[simp]
theorem cocompact_map.comp_id {α : Type u_1} {β : Type u_2} [topological_space α] [topological_space β] (f : cocompact_map α β) :
theorem cocompact_map.is_compact_preimage {α : Type u_1} {β : Type u_2} [topological_space α] [topological_space β] [t2_space β] (f : cocompact_map α β) ⦃s : set β⦄ (hs : is_compact s) :

If the codomain is Hausdorff, preimages of compact sets are compact under a cocompact continuous map.

def homeomorph.to_cocompact_map {α : Type u_1} {β : Type u_2} [topological_space α] [topological_space β] (f : α ≃ₜ β) :

A homemomorphism is a cocompact map.

Equations
@[simp]