Compact sets and compact spaces #
Main definitions #
We define the following properties for sets in a topological space:
IsCompact
: a set such that each open cover has a finite subcover. This is defined in mathlib using filters. The main property of a compact set isIsCompact.elim_finite_subcover
.CompactSpace
: typeclass stating that the whole space is a compact set.NoncompactSpace
: a space that is not a compact space.
Main results #
isCompact_univ_pi
: Tychonov's theorem - an arbitrary product of compact sets is compact.
The complement to a compact set belongs to a filter f
if each x ∈ s
has a neighborhood t
within s
such that tᶜ
belongs to f
.
If p : Set X → Prop
is stable under restriction and union, and each point x
of a compact set s
has a neighborhood t
within s
such that p t
, then p s
holds.
The intersection of a compact set and a closed set is a compact set.
The intersection of a closed set and a compact set is a compact set.
The set difference of a compact set and an open set is a compact set.
A closed subset of a compact set is a compact set.
Alias of the forward direction of isCompact_iff_ultrafilter_le_nhds
.
Alias of the forward direction of isCompact_iff_ultrafilter_le_nhds'
.
If a compact set belongs to a filter and this filter has a unique cluster point y
in this set,
then the filter is less than or equal to 𝓝 y
.
If values of f : Y → X
belong to a compact set s
eventually along a filter l
and y
is a unique MapClusterPt
for f
along l
in s
,
then f
tends to 𝓝 y
along l
.
For every open directed cover of a compact set, there exists a single element of the cover which itself includes the set.
For every open cover of a compact set, there exists a finite subcover.
The neighborhood filter of a compact set is disjoint with a filter l
if and only if the
neighborhood filter of each point of this set is disjoint with l
.
A filter l
is disjoint with the neighborhood filter of a compact set if and only if it is
disjoint with the neighborhood filter of each point of this set.
For every directed family of closed sets whose intersection avoids a compact set, there exists a single element of the family which itself avoids this compact set.
For every family of closed sets whose intersection avoids a compact set, there exists a finite subfamily whose intersection avoids this compact set.
If s
is a compact set in a topological space X
and f : ι → Set X
is a locally finite
family of sets, then f i ∩ s
is nonempty only for a finitely many i
.
To show that a compact set intersects the intersection of a family of closed sets, it is sufficient to show that it intersects every finite subfamily.
Cantor's intersection theorem for iInter
:
the intersection of a directed family of nonempty compact closed sets is nonempty.
Alias of IsCompact.nonempty_iInter_of_directed_nonempty_isCompact_isClosed
.
Cantor's intersection theorem for iInter
:
the intersection of a directed family of nonempty compact closed sets is nonempty.
Cantor's intersection theorem for sInter
:
the intersection of a directed family of nonempty compact closed sets is nonempty.
Cantor's intersection theorem for sequences indexed by ℕ
:
the intersection of a decreasing sequence of nonempty compact closed sets is nonempty.
Alias of IsCompact.nonempty_iInter_of_sequence_nonempty_isCompact_isClosed
.
Cantor's intersection theorem for sequences indexed by ℕ
:
the intersection of a decreasing sequence of nonempty compact closed sets is nonempty.
For every open cover of a compact set, there exists a finite subcover.
A set s
is compact if for every open cover of s
, there exists a finite subcover.
A set s
is compact if for every family of closed sets whose intersection avoids s
,
there exists a finite subfamily whose intersection avoids s
.
A set s
is compact if and only if
for every open cover of s
, there exists a finite subcover.
A set s
is compact if and only if
for every family of closed sets whose intersection avoids s
,
there exists a finite subfamily whose intersection avoids s
.
If s : Set (X × Y)
belongs to 𝓝 x ×ˢ l
for all x
from a compact set K
,
then it belongs to (𝓝ˢ K) ×ˢ l
,
i.e., there exist an open U ⊇ K
and t ∈ l
such that U ×ˢ t ⊆ s
.
If s : Set (X × Y)
belongs to l ×ˢ 𝓝 y
for all y
from a compact set K
,
then it belongs to l ×ˢ (𝓝ˢ K)
,
i.e., there exist t ∈ l
and an open U ⊇ K
such that t ×ˢ U ⊆ s
.
If s : Set X
belongs to 𝓝 x ⊓ l
for all x
from a compact set K
,
then it belongs to (𝓝ˢ K) ⊓ l
,
i.e., there exist an open U ⊇ K
and T ∈ l
such that U ∩ T ⊆ s
.
If s : Set S
belongs to l ⊓ 𝓝 x
for all x
from a compact set K
,
then it belongs to l ⊓ (𝓝ˢ K)
,
i.e., there exist T ∈ l
and an open U ⊇ K
such that T ∩ U ⊆ s
.
To show that ∀ y ∈ K, P x y
holds for x
close enough to x₀
when K
is compact,
it is sufficient to show that for all y₀ ∈ K
there P x y
holds for (x, y)
close enough
to (x₀, y₀)
.
Provided for backwards compatibility,
see IsCompact.mem_prod_nhdsSet_of_forall
for a stronger statement.
If V : ι → Set X
is a decreasing family of closed compact sets then any neighborhood of
⋂ i, V i
contains some V i
. We assume each V i
is compact and closed because X
is
not assumed to be Hausdorff. See exists_subset_nhd_of_compact
for version assuming this.
If X
has a basis consisting of compact opens, then an open set in X
is compact open iff
it is a finite union of some elements in the basis
A filter is disjoint from the cocompact filter if and only if it contains a compact set.
A filter is disjoint from the cocompact filter if and only if it contains a compact set.
A set belongs to coclosedCompact
if and only if the closure of its complement is compact.
Complement of a set belongs to coclosedCompact
if and only if its closure is compact.
Sets that are contained in a compact set form a bornology. Its cobounded
filter is
Filter.cocompact
. See also Bornology.relativelyCompact
the bornology of sets with compact
closure.
Equations
- Bornology.inCompact X = { cobounded' := Filter.cocompact X, le_cofinite' := ⋯ }
Instances For
If s
and t
are compact sets, then the set neighborhoods filter of s ×ˢ t
is the product of set neighborhoods filters for s
and t
.
For general sets, only the ≤
inequality holds, see nhdsSet_prod_le
.
If s
and t
are compact sets and n
is an open neighborhood of s × t
, then there exist
open neighborhoods u ⊇ s
and v ⊇ t
such that u × v ⊆ n
.
See also IsCompact.nhdsSet_prod_eq
.
If a filter has a unique cluster point y
in a compact topological space,
then the filter is less than or equal to 𝓝 y
.
If y
is a unique MapClusterPt
for f
along l
and the codomain of f
is a compact space,
then f
tends to 𝓝 y
along l
.
A compact discrete space is finite.
If X
is a compact space, then a locally finite family of sets of X
can have only finitely
many nonempty elements.
If X
is a compact space, then a locally finite family of nonempty sets of X
can have only
finitely many elements, Set.Finite
version.
If X
is a compact space, then a locally finite family of nonempty sets of X
can have only
finitely many elements, Fintype
version.
Equations
- hf.fintypeOfCompact hne = Set.fintypeOfFiniteUniv ⋯
Instances For
The comap of the cocompact filter on Y
by a continuous function f : X → Y
is less than or
equal to the cocompact filter on X
.
This is a reformulation of the fact that images of compact sets are compact.
If a filter is disjoint from the cocompact filter, so is its image under any continuous function.
If X
is a compact topological space, then Prod.snd : X × Y → Y
is a closed map.
If Y
is a compact topological space, then Prod.fst : X × Y → X
is a closed map.
If f : X → Y
is an inducing map, the image f '' s
of a set s
is compact
if and only if s
is compact.
Alias of Topology.IsInducing.isCompact_iff
.
If f : X → Y
is an inducing map, the image f '' s
of a set s
is compact
if and only if s
is compact.
If f : X → Y
is an Embedding
, the image f '' s
of a set s
is compact
if and only if s
is compact.
Alias of Topology.IsEmbedding.isCompact_iff
.
If f : X → Y
is an Embedding
, the image f '' s
of a set s
is compact
if and only if s
is compact.
The preimage of a compact set under an inducing map is a compact set.
Alias of Topology.IsInducing.isCompact_preimage
.
The preimage of a compact set under an inducing map is a compact set.
The preimage of a compact set in the image of an inducing map is compact.
Alias of Topology.IsInducing.isCompact_preimage'
.
The preimage of a compact set in the image of an inducing map is compact.
The preimage of a compact set under a closed embedding is a compact set.
Alias of Topology.IsClosedEmbedding.isCompact_preimage
.
The preimage of a compact set under a closed embedding is a compact set.
A closed embedding is proper, ie, inverse images of compact sets are contained in compacts.
Moreover, the preimage of a compact set is compact, see IsClosedEmbedding.isCompact_preimage
.
Alias of Topology.IsClosedEmbedding.tendsto_cocompact
.
A closed embedding is proper, ie, inverse images of compact sets are contained in compacts.
Moreover, the preimage of a compact set is compact, see IsClosedEmbedding.isCompact_preimage
.
Sets of subtype are compact iff the image under a coercion is.
Alias of Topology.IsClosedEmbedding.compactSpace
.
Finite topological spaces are compact.
The product of two compact spaces is compact.
The disjoint union of two compact spaces is compact.
The coproduct of the cocompact filters on two topological spaces is the cocompact filter on their product.
Tychonoff's theorem: product of compact sets is compact.
Tychonoff's theorem formulated using Set.pi
: product of compact sets is compact.
Tychonoff's theorem formulated in terms of filters: Filter.cocompact
on an indexed product
type Π d, X d
the Filter.coprodᵢ
of filters Filter.cocompact
on X d
.