Sequences in topological spaces #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
In this file we define sequences in topological spaces and show how they are related to filters and the topology.
Main definitions #
Set operation #
seq_closure s
: sequential closure of a set, the set of limits of sequences of points ofs
;
Predicates #
is_seq_closed s
: predicate saying that a set is sequentially closed, i.e.,seq_closure s ⊆ s
;seq_continuous f
: predicate saying that a function is sequentially continuous, i.e., for any sequenceu : ℕ → X
that converges to a pointx
, the sequencef ∘ u
converges tof x
;is_seq_compact s
: predicate saying that a set is sequentially compact, i.e., every sequence taking values ins
has a converging subsequence.
Type classes #
frechet_urysohn_space X
: a typeclass saying that a topological space is a Fréchet-Urysohn space, i.e., the sequential closure of any set is equal to its closure.sequential_space X
: a typeclass saying that a topological space is a sequential space, i.e., any sequentially closed set in this space is closed. This condition is weaker than being a Fréchet-Urysohn space.seq_compact_space X
: a typeclass saying that a topological space is sequentially compact, i.e., every sequence inX
has a converging subsequence.
Main results #
seq_closure_subset_closure
: closure of a set includes its sequential closure;is_closed.is_seq_closed
: a closed set is sequentially closed;is_seq_closed.seq_closure_eq
: sequential closure of a sequentially closed sets
is equal tos
;seq_closure_eq_closure
: in a Fréchet-Urysohn space, the sequential closure of a set is equal to its closure;tendsto_nhds_iff_seq_tendsto
,frechet_urysohn_space.of_seq_tendsto_imp_tendsto
: a topological space is a Fréchet-Urysohn space if and only if sequential convergence implies convergence;topological_space.first_countable_topology.frechet_urysohn_space
: every topological space with first countable topology is a Fréchet-Urysohn space;frechet_urysohn_space.to_sequential_space
: every Fréchet-Urysohn space is a sequential space;is_seq_compact.is_compact
: a sequentially compact set in a uniform space with countably generated uniformity is compact.
Tags #
sequentially closed, sequentially compact, sequential space
Sequential closures, sequential continuity, and sequential spaces. #
The sequential closure of a set s : set X
in a topological space X
is the set of all a : X
which arise as limit of sequences in s
. Note that the sequential closure of a set is not
guaranteed to be sequentially closed.
Equations
- seq_closure s = {a : X | ∃ (x : ℕ → X), (∀ (n : ℕ), x n ∈ s) ∧ filter.tendsto x filter.at_top (nhds a)}
The sequential closure of a set is contained in the closure of that set. The converse is not true.
A set s
is sequentially closed if for any converging sequence x n
of elements of s
, the
limit belongs to s
as well. Note that the sequential closure of a set is not guaranteed to be
sequentially closed.
Equations
- is_seq_closed s = ∀ ⦃x : ℕ → X⦄ ⦃p : X⦄, (∀ (n : ℕ), x n ∈ s) → filter.tendsto x filter.at_top (nhds p) → p ∈ s
The sequential closure of a sequentially closed set is the set itself.
If a set is equal to its sequential closure, then it is sequentially closed.
A set is sequentially closed iff it is equal to its sequential closure.
A set is sequentially closed if it is closed.
- closure_subset_seq_closure : ∀ (s : set X), closure s ⊆ seq_closure s
A topological space is called a Fréchet-Urysohn space, if the sequential closure of any set is equal to its closure. Since one of the inclusions is trivial, we require only the non-trivial one in the definition.
Instances of this typeclass
In a Fréchet-Urysohn space, a point belongs to the closure of a set iff it is a limit of a sequence taking values in this set.
If the domain of a function f : α → β
is a Fréchet-Urysohn space, then convergence
is equivalent to sequential convergence. See also filter.tendsto_iff_seq_tendsto
for a version
that works for any pair of filters assuming that the filter in the domain is countably generated.
This property is equivalent to the definition of frechet_urysohn_space
, see
frechet_urysohn_space.of_seq_tendsto_imp_tendsto
.
An alternative construction for frechet_urysohn_space
: if sequential convergence implies
convergence, then the space is a Fréchet-Urysohn space.
Every first-countable space is a Fréchet-Urysohn space.
- is_closed_of_seq : ∀ (s : set X), is_seq_closed s → is_closed s
A topological space is said to be a sequential space if any sequentially closed set in this space is closed. This condition is weaker than being a Fréchet-Urysohn space.
Instances of this typeclass
Every Fréchet-Urysohn space is a sequential space.
In a sequential space, a sequentially closed set is closed.
In a sequential space, a set is closed iff it's sequentially closed.
A function between topological spaces is sequentially continuous if it commutes with limit of convergent sequences.
Equations
- seq_continuous f = ∀ ⦃x : ℕ → X⦄ ⦃p : X⦄, filter.tendsto x filter.at_top (nhds p) → filter.tendsto (f ∘ x) filter.at_top (nhds (f p))
The preimage of a sequentially closed set under a sequentially continuous map is sequentially closed.
A sequentially continuous function defined on a sequential space is continuous.
If the domain of a function is a sequential space, then continuity of this function is equivalent to its sequential continuity.
The quotient of a sequential space is a sequential space.
A set s
is sequentially compact if every sequence taking values in s
has a
converging subsequence.
- seq_compact_univ : is_seq_compact set.univ
A space X
is sequentially compact if every sequence in X
has a
converging subsequence.
Instances of this typeclass
A sequentially compact set in a uniform space is totally bounded.
A sequentially compact set in a uniform set with countably generated uniformity filter is complete.
If 𝓤 β
is countably generated, then any sequentially compact set is compact.
A version of Bolzano-Weistrass: in a uniform space with countably generated uniformity filter (e.g., in a metric space), a set is compact if and only if it is sequentially compact.
A version of Bolzano-Weistrass: in a proper metric space (eg. $ℝ^n$), every bounded sequence has a converging subsequence. This version assumes only that the sequence is frequently in some bounded set.
A version of Bolzano-Weistrass: in a proper metric space (eg. $ℝ^n$), every bounded sequence has a converging subsequence.