The OnePoint Compactification #
We construct the OnePoint compactification (the one-point compactification) of an arbitrary
topological space X and prove some properties inherited from X.
Main definitions #
OnePoint: the OnePoint compactification, we use coercion for the canonical embeddingX → OnePoint X; whenXis already compact, the compactification adds an isolated point to the space.OnePoint.infty: the extra point
Main results #
- The topological structure of
OnePoint X - The connectedness of
OnePoint Xfor a noncompact, preconnectedX OnePoint XisT₀for a T₀ spaceXOnePoint XisT₁for a T₁ spaceXOnePoint Xis normal ifXis a locally compact Hausdorff space
Tags #
one-point compactification, Alexandroff compactification, compactness
Definition and basic properties #
In this section we define OnePoint X to be the disjoint union of X and ∞, implemented as
Option X. Then we restate some lemmas about Option X for OnePoint X.
The repr uses the notation from the OnePoint locale.
Equations
- instReprOnePoint = { reprPrec := fun (o : OnePoint X) (x : ℕ) => match o with | none => Std.Format.text "∞" | some a => Std.Format.text "↑" ++ repr a }
The point at infinity
Equations
Instances For
The point at infinity
Equations
- OnePoint.«term∞» = Lean.ParserDescr.node `OnePoint.«term∞» 1024 (Lean.ParserDescr.symbol "∞")
Instances For
Equations
- OnePoint.instCoeTC = { coe := OnePoint.some }
Equations
- OnePoint.instInhabited = { default := OnePoint.infty }
Equations
Recursor for OnePoint using the preferred forms ∞ and ↑x.
Equations
- OnePoint.rec infty coe none = infty
- OnePoint.rec infty coe (some a) = coe a
Instances For
Alias of OnePoint.notMem_range_coe_iff.
Alias of OnePoint.infty_notMem_range_coe.
Alias of OnePoint.infty_notMem_image_coe.
Extend a map f : X → Y to a map OnePoint X → OnePoint Y
by sending infinity to infinity.
Equations
- OnePoint.map f = Option.map f
Instances For
Topological space structure on OnePoint X #
We define a topological space structure on OnePoint X so that s is open if and only if
(↑) ⁻¹' sis open inX;- if
∞ ∈ s, then((↑) ⁻¹' s)ᶜis compact.
Then we reformulate this definition in a few different ways, and prove that
(↑) : X → OnePoint X is an open embedding. If X is not a compact space, then we also prove
that (↑) has dense range, so it is a dense embedding.
Equations
- One or more equations did not get rendered due to their size.
Alias of OnePoint.isOpen_iff_of_notMem.
An open set in OnePoint X constructed from a closed compact set in X
Equations
- OnePoint.opensOfCompl s h₁ h₂ = { carrier := (OnePoint.some '' s)ᶜ, is_open' := ⋯ }
Instances For
If x is not an isolated point of X, then x : OnePoint X is not an isolated point
of OnePoint X.
Alias of OnePoint.nhdsNE_coe_neBot.
If x is not an isolated point of X, then x : OnePoint X is not an isolated point
of OnePoint X.
Alias of OnePoint.nhdsNE_infty_eq.
If X is a non-compact space, then ∞ is not an isolated point of OnePoint X.
Alias of OnePoint.nhdsNE_infty_neBot.
If X is a non-compact space, then ∞ is not an isolated point of OnePoint X.
Alias of OnePoint.nhdsNE_neBot.
A constructor for continuous maps out of a one point compactification, given a continuous map from the underlying space and a limit value at infinity.
Equations
Instances For
A constructor for continuous maps out of a one point compactification of a discrete space, given a map from the underlying space and a limit value at infinity.
Equations
- OnePoint.continuousMapMkDiscrete f y h = OnePoint.continuousMapMk { toFun := f, continuous_toFun := ⋯ } y ⋯
Instances For
Continuous maps out of the one point compactification of an infinite discrete space to a Hausdorff space correspond bijectively to "convergent" maps out of the discrete space.
Equations
- One or more equations did not get rendered due to their size.
Instances For
A constructor for continuous maps out of the one point compactification of ℕ, given a
sequence and a limit value at infinity.
Equations
Instances For
Continuous maps out of the one point compactification of ℕ to a Hausdorff space Y correspond
bijectively to convergent sequences in Y.
Equations
- One or more equations did not get rendered due to their size.
Instances For
If X is not a compact space, then the natural embedding X → OnePoint X has dense range.
Compactness and separation properties #
In this section we prove that OnePoint X is a compact space; it is a T₀ (resp., T₁) space if
the original space satisfies the same separation axiom. If the original space is a locally compact
Hausdorff space, then OnePoint X is a normal (hence, T₃ and Hausdorff) space.
Finally, if the original space X is not compact and is a preconnected space, then
OnePoint X is a connected space.
For any topological space X, its one point compactification is a compact space.
The one point compactification of a weakly locally compact R₁ space is a normal topological space.
If X is not a compact space, then OnePoint X is a connected space.
If X is an infinite type with discrete topology (e.g., ℕ), then the identity map from
CofiniteTopology (OnePoint X) to OnePoint X is not continuous.
If f embeds X into a compact Hausdorff space Y, and has exactly one point outside its
range, then (Y, f) is the one-point compactification of X.
Equations
Instances For
Extend a homeomorphism of topological spaces to the homeomorphism of their one point compactifications.
Equations
- h.onePointCongr = { toFun := OnePoint.map ⇑h, invFun := OnePoint.map ⇑h.symm, left_inv := ⋯, right_inv := ⋯, continuous_toFun := ⋯, continuous_invFun := ⋯ }
Instances For
A concrete counterexample shows that Continuous.homeoOfEquivCompactToT2
cannot be generalized from T2Space to T1Space.
Let α = OnePoint ℕ be the one-point compactification of ℕ, and let β be the same space
OnePoint ℕ with the cofinite topology. Then α is compact, β is T1, and the identity map
id : α → β is a continuous equivalence that is not a homeomorphism.