Sequences in topological spaces
In this file we define sequences in topological spaces and show how they are related to filters and the topology. In particular, we
- define the sequential closure of a set and prove that it's contained in the closure,
- define a type class "sequential_space" in which closure and sequential closure agree,
- define sequential continuity and show that it coincides with continuity in sequential spaces,
- provide an instance that shows that every first-countable (and in particular metric) space is a sequential space.
- define sequential compactness, prove that compactness implies sequential compactness in first countable spaces, and prove they are equivalent for uniform spaces having a countable uniformity basis (in particular metric spaces).
Sequential closures, sequential continuity, and sequential spaces.
A sequence converges in the sence of topological spaces iff the associated statement for filter holds.
The sequential closure of a subset M ⊆ α of a topological space α is the set of all p ∈ α which arise as limit of sequences in M.
Equations
- sequential_closure M = {p : α | ∃ (x : ℕ → α), (∀ (n : ℕ), x n ∈ M) ∧ filter.tendsto x filter.at_top (nhds p)}
A set s
is sequentially closed if for any converging sequence x n
of elements of s
,
the limit belongs to s
as well.
Equations
- is_seq_closed s = (s = sequential_closure s)
A convenience lemma for showing that a set is sequentially closed.
The sequential closure of a set is contained in the closure of that set. The converse is not true.
A set is sequentially closed if it is closed.
The limit of a convergent sequence in a sequentially closed set is in that set.
The limit of a convergent sequence in a closed set is in that set.
- sequential_closure_eq_closure : ∀ (M : set α), sequential_closure M = closure M
A sequential space is a space in which 'sequences are enough to probe the topology'. This can be formalised by demanding that the sequential closure and the closure coincide. The following statements show that other topological properties can be deduced from sequences in sequential spaces.
In a sequential space, a set is closed iff it's sequentially closed.
In a sequential space, a point belongs to the closure of a set iff it is a limit of a sequence taking values in this set.
A function between topological spaces is sequentially continuous if it commutes with limit of convergent sequences.
Equations
- sequentially_continuous f = ∀ (x : ℕ → α) {limit : α}, filter.tendsto x filter.at_top (nhds limit) → filter.tendsto (f ∘ x) filter.at_top (nhds (f limit))
In a sequential space, continuity and sequential continuity coincide.
Every first-countable space is sequential.
Equations
A set s
is sequentially compact if every sequence taking values in s
has a
converging subsequence.
Equations
- is_seq_compact s = ∀ ⦃u : ℕ → α⦄, (∀ (n : ℕ), u n ∈ s) → (∃ (x : α) (H : x ∈ s) (φ : ℕ → ℕ), strict_mono φ ∧ filter.tendsto (u ∘ φ) filter.at_top (nhds x))
- seq_compact_univ : is_seq_compact set.univ
A space α
is sequentially compact if every sequence in α
has a
converging subsequence.
Equations
A version of Bolzano-Weistrass: in a metric space, is_compact s ↔ is_seq_compact s
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.