mathlib documentation

topology.​sequences

topology.​sequences

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

Sequential closures, sequential continuity, and sequential spaces.

theorem topological_space.​seq_tendsto_iff {α : Type u_1} [topological_space α] {x : → α} {limit : α} :
filter.tendsto x filter.at_top (nhds limit) ∀ (U : set α), limit Uis_open U(∃ (N : ), ∀ (n : ), n Nx n U)

A sequence converges in the sence of topological spaces iff the associated statement for filter holds.

def sequential_closure {α : Type u_1} [topological_space α] :
set αset α

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
theorem subset_sequential_closure {α : Type u_1} [topological_space α] (M : set α) :

def is_seq_closed {α : Type u_1} [topological_space α] :
set α → Prop

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
theorem is_seq_closed_of_def {α : Type u_1} [topological_space α] {A : set α} :
(∀ (x : → α) (p : α), (∀ (n : ), x n A)filter.tendsto x filter.at_top (nhds p)p A)is_seq_closed A

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.

theorem is_seq_closed_of_is_closed {α : Type u_1} [topological_space α] (M : set α) :

A set is sequentially closed if it is closed.

theorem mem_of_is_seq_closed {α : Type u_1} [topological_space α] {A : set α} (_x : is_seq_closed A) {x : → α} (_x_1 : ∀ (n : ), x n A) {limit : α} :
filter.tendsto x filter.at_top (nhds limit)limit A

The limit of a convergent sequence in a sequentially closed set is in that set.

theorem mem_of_is_closed_sequential {α : Type u_1} [topological_space α] {A : set α} (_x : is_closed A) {x : → α} (_x_1 : ∀ (n : ), x n A) {limit : α} :
filter.tendsto x filter.at_top (nhds limit)limit A

The limit of a convergent sequence in a closed set is in that set.

@[class]
structure sequential_space (α : Type u_3) [topological_space α] :
Prop

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.

Instances

In a sequential space, a set is closed iff it's sequentially closed.

theorem mem_closure_iff_seq_limit {α : Type u_1} [topological_space α] [sequential_space α] {s : set α} {a : α} :
a closure s ∃ (x : → α), (∀ (n : ), x n s) filter.tendsto x filter.at_top (nhds a)

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.

def sequentially_continuous {α : Type u_1} {β : Type u_2} [topological_space α] [topological_space β] :
(α → β) → Prop

A function between topological spaces is sequentially continuous if it commutes with limit of convergent sequences.

Equations
theorem continuous.​to_sequentially_continuous {α : Type u_1} {β : Type u_2} [topological_space α] [topological_space β] {f : α → β} :

theorem continuous_iff_sequentially_continuous {α : Type u_1} {β : Type u_2} [topological_space α] [topological_space β] {f : α → β} [sequential_space α] :

In a sequential space, continuity and sequential continuity coincide.

def is_seq_compact {α : Type u_1} [topological_space α] :
set α → Prop

A set s is sequentially compact if every sequence taking values in s has a converging subsequence.

Equations
@[class]
structure seq_compact_space (α : Type u_3) [topological_space α] :
Prop

A space α is sequentially compact if every sequence in α has a converging subsequence.

Instances
theorem is_seq_compact.​subseq_of_frequently_in {α : Type u_1} [topological_space α] {s : set α} (hs : is_seq_compact s) {u : → α} :
(∃ᶠ (n : ) in filter.at_top, u n s)(∃ (x : α) (H : x s) (φ : ), strict_mono φ filter.tendsto (u φ) filter.at_top (nhds x))

theorem seq_compact_space.​tendsto_subseq {α : Type u_1} [topological_space α] [seq_compact_space α] (u : → α) :
∃ (x : α) (φ : ), strict_mono φ filter.tendsto (u φ) filter.at_top (nhds x)

theorem is_compact.​tendsto_subseq' {α : Type u_1} [topological_space α] [topological_space.first_countable_topology α] {s : set α} {u : → α} :
is_compact s(∃ᶠ (n : ) in filter.at_top, u n s)(∃ (x : α) (H : x s) (φ : ), strict_mono φ filter.tendsto (u φ) filter.at_top (nhds x))

theorem is_compact.​tendsto_subseq {α : Type u_1} [topological_space α] [topological_space.first_countable_topology α] {s : set α} {u : → α} :
is_compact s(∀ (n : ), u n s)(∃ (x : α) (H : x s) (φ : ), strict_mono φ filter.tendsto (u φ) filter.at_top (nhds x))

theorem lebesgue_number_lemma_seq {β : Type u_2} [uniform_space β] {s : set β} {ι : Type u_1} {c : ι → set β} :
is_seq_compact s(∀ (i : ι), is_open (c i))(s ⋃ (i : ι), c i)(uniformity β).is_countably_generated(∃ (V : set × β)) (H : V uniformity β), symmetric_rel V ∀ (x : β), x s(∃ (i : ι), uniform_space.ball x V c i))

theorem is_seq_compact.​totally_bounded {β : Type u_2} [uniform_space β] {s : set β} :

theorem metric.​compact_iff_seq_compact {β : Type u_2} [metric_space β] {s : set β} :

A version of Bolzano-Weistrass: in a metric space, is_compact s ↔ is_seq_compact s

theorem tendsto_subseq_of_frequently_bounded {β : Type u_2} [metric_space β] {s : set β} [proper_space β] (hs : metric.bounded s) {u : → β} :
(∃ᶠ (n : ) in filter.at_top, u n s)(∃ (b : β) (H : b closure s) (φ : ), strict_mono φ filter.tendsto (u φ) filter.at_top (nhds b))

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.

theorem tendsto_subseq_of_bounded {β : Type u_2} [metric_space β] {s : set β} [proper_space β] (hs : metric.bounded s) {u : → β} :
(∀ (n : ), u n s)(∃ (b : β) (H : b closure s) (φ : ), strict_mono φ filter.tendsto (u φ) filter.at_top (nhds b))

A version of Bolzano-Weistrass: in a proper metric space (eg. $ℝ^n$), every bounded sequence has a converging subsequence.

theorem seq_compact.​lebesgue_number_lemma_of_metric {β : Type u_2} [metric_space β] {s : set β} {ι : Type u_1} {c : ι → set β} :
is_seq_compact s(∀ (i : ι), is_open (c i))(s ⋃ (i : ι), c i)(∃ (δ : ) (H : δ > 0), ∀ (x : β), x s(∃ (i : ι), metric.ball x δ c i))