A T₀ space, also known as a Kolmogorov space, is a topological space
where for every pair x ≠ y
, there is an open set containing one but not the other.
Instances
- t1 : ∀ (x : α), is_closed {x}
A T₁ space, also known as a Fréchet space, is a topological space
where every singleton set is closed. Equivalently, for every pair
x ≠ y
, there is an open set containing x
and not y
.
A T₂ space, also known as a Hausdorff space, is one in which for every
x ≠ y
there exists disjoint open sets around x
and y
. This is
the most widely used of the separation axioms.
Properties of Lim
and lim
In this section we use explicit nonempty α
instances for Lim
and lim
. This way the lemmas
are useful without a nonempty α
instance.
If a compact set is covered by two open sets, then we can cover it by two compact subsets.
For every finite open cover Uᵢ
of a compact set, there exists a compact cover Kᵢ ⊆ Uᵢ
.
In a locally compact T₂ space, every point has an open neighborhood with compact closure
In a locally compact T₂ space, every compact set is contained in the interior of a compact set.
- to_t1_space : t1_space α
- regular : ∀ {s : set α} {a : α}, is_closed s → a ∉ s → (∃ (t : set α), is_open t ∧ s ⊆ t ∧ 𝓝[t] a = ⊥)
A T₃ space, also known as a regular space (although this condition sometimes
omits T₂), is one in which for every closed C
and x ∉ C
, there exist
disjoint open sets containing x
and C
respectively.
- to_t1_space : t1_space α
- normal : ∀ (s t : set α), is_closed s → is_closed t → disjoint s t → (∃ (u v : set α), is_open u ∧ is_open v ∧ s ⊆ u ∧ t ⊆ v ∧ disjoint u v)
A T₄ space, also known as a normal space (although this condition sometimes
omits T₂), is one in which for every pair of disjoint closed sets C
and D
,
there exist disjoint open sets containing C
and D
respectively.