Skip to content

Instantly share code, notes, and snippets.

@PatrickMassot
Last active September 9, 2018 21:41
Show Gist options
  • Star 1 You must be signed in to star a gist
  • Fork 0 You must be signed in to fork a gist
  • Save PatrickMassot/1b2d39011855ba43f3bf00c08051ad9e to your computer and use it in GitHub Desktop.
Save PatrickMassot/1b2d39011855ba43f3bf00c08051ad9e to your computer and use it in GitHub Desktop.
import analysis.metric_space
variables {α : Type*} [metric_space α] {β : Type*}
open filter
lemma tendsto_nhds_iff (u : β → α) (f : filter β) (a : α) : tendsto u f (nhds a) ↔
∀ ε > 0, {n | dist (u n) a < ε} ∈ f.sets :=
⟨λ H ε εpos, H (ball_mem_nhds a εpos),
λ H s s_nhd, let ⟨ε, εpos, sub⟩ := mem_nhds_iff_metric.1 s_nhd in
f.sets_of_superset (H ε εpos) (λ b b_in, sub b_in)⟩
lemma seq_tendsto_iff (u : ℕ → α) (a : α) : tendsto u at_top (nhds a) ↔
∀ ε > 0, ∃ (N : ℕ), ∀ {n}, n ≥ N → dist (u n) a < ε :=
by simp [tendsto_nhds_iff, mem_at_top_sets]
Sign up for free to join this conversation on GitHub. Already have an account? Sign in to comment