Zulip Chat Archive
Stream: new members
Topic: Show tails of a convergent sequence converge
mdnestor (Aug 06 2024 at 01:20):
Hi, I am trying to show the tails of a convergent sequence also converge, any ideas? The mathlib docs on theorems about filters is greek to me :)
import Mathlib.Topology.Basic
def converge [TopologicalSpace X] (a: Nat → X) (x: X): Prop :=
Filter.Tendsto a Filter.atTop (nhds x)
theorem tails_converge [TopologicalSpace X] {a: Nat → X} {x: X} (h: converge a x): ∀ t: Nat, converge (a ∘ (fun n => n + t)) x := by
sorry
mdnestor (Aug 06 2024 at 03:15):
This is pretty easy using standard topological definition of convergent sequence but I also cannot find the equivalence to the filter definition
Jireh Loreaux (Aug 06 2024 at 03:28):
@loogle HAdd.hAdd, Nat, Filter.Tendsto, Filter.atTop
loogle (Aug 06 2024 at 03:28):
:search: Filter.tendsto_add_atTop_nat, Filter.tendsto_add_atTop_iff_nat, and 62 more
Jireh Loreaux (Aug 06 2024 at 03:30):
How about docs#Filter.Tendsto.comp + docs#Filter.tendsto_add_atTop_nat ?
Jireh Loreaux (Aug 06 2024 at 03:31):
You should read #mil if you don't understand filters.
Jireh Loreaux (Aug 06 2024 at 03:32):
Namely, starting with Section 9.1
mdnestor (Aug 07 2024 at 20:22):
So the theorem I was looking for is tendsto_atTop_nhds
which is the equivalence between the filter definition of convergent sequence and the standard topological definition. Here is complete proof.
import Mathlib.Topology.Basic
def converge [TopologicalSpace X] (a: Nat → X) (x: X): Prop :=
Filter.Tendsto a Filter.atTop (nhds x)
theorem tails_converge [TopologicalSpace X] {a: Nat → X} {x: X} (h: converge a x): ∀ t: Nat, converge (a ∘ (fun n => n + t)) x := by
intro t
rw [converge, tendsto_atTop_nhds]
have h1 := tendsto_atTop_nhds.mp h
intro U hx hU
obtain ⟨N, hN⟩ := h1 U hx hU
exists N - t
intro n h2
simp at h2
exact hN (n + t) h2
Luigi Massacci (Aug 08 2024 at 08:59):
This way you are doing the proof "manually" (which might be what you want of course), but the two lemmas Jireh suggested to you should suffice to one-line it
Last updated: May 02 2025 at 03:31 UTC