Convergence to infinity and countably generated filters #
In this file we prove that
Filter.atTop
andFilter.atBot
filters on a countable type are countably generated;Filter.exists_seq_tendsto
: iff
is a nontrivial countably generated filter, then there exists a sequence that converges. tof
;Filter.tendsto_iff_seq_tendsto
: convergence along a countably generated filter is equivalent to convergence along all sequences that converge to this filter.
instance
OrderDual.instIsCountablyGeneratedAtTop
{α : Type u_1}
[Preorder α]
[Filter.atBot.IsCountablyGenerated]
:
Filter.atTop.IsCountablyGenerated
instance
OrderDual.instIsCountablyGeneratedAtBot
{α : Type u_1}
[Preorder α]
[Filter.atTop.IsCountablyGenerated]
:
Filter.atBot.IsCountablyGenerated
theorem
Filter.tendsto_iff_seq_tendsto
{α : Type u_1}
{β : Type u_2}
{f : α → β}
{k : Filter α}
{l : Filter β}
[k.IsCountablyGenerated]
:
An abstract version of continuity of sequentially continuous functions on metric spaces:
if a filter k
is countably generated then Tendsto f k l
iff for every sequence u
converging to k
, f ∘ u
tends to l
.
theorem
Filter.tendsto_of_subseq_tendsto
{α : Type u_1}
{ι : Type u_3}
{x : ι → α}
{f : Filter α}
{l : Filter ι}
[l.IsCountablyGenerated]
(hxy : ∀ (ns : ℕ → ι), Tendsto ns atTop l → ∃ (ms : ℕ → ℕ), Tendsto (fun (n : ℕ) => x (ns (ms n))) atTop f)
:
Tendsto x l f
A sequence converges if every subsequence has a convergent subsequence.