mathlib3 documentation

topology.uniform_space.uniform_convergence

Uniform convergence #

THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.

A sequence of functions Fₙ (with values in a metric space) converges uniformly on a set s to a function f if, for all ε > 0, for all large enough n, one has for all y ∈ s the inequality dist (f y, Fₙ y) < ε. Under uniform convergence, many properties of the Fₙ pass to the limit, most notably continuity. We prove this in the file, defining the notion of uniform convergence in the more general setting of uniform spaces, and with respect to an arbitrary indexing set endowed with a filter (instead of just with at_top).

Main results #

Let α be a topological space, β a uniform space, Fₙ and f be functions from αto β (where the index n belongs to an indexing type ι endowed with a filter p).

We also define notions where the convergence is locally uniform, called tendsto_locally_uniformly_on F f p s and tendsto_locally_uniformly F f p. The previous theorems all have corresponding versions under locally uniform convergence.

Finally, we introduce the notion of a uniform Cauchy sequence, which is to uniform convergence what a Cauchy sequence is to the usual notion of convergence.

Implementation notes #

We derive most of our initial results from an auxiliary definition tendsto_uniformly_on_filter. This definition in and of itself can sometimes be useful, e.g., when studying the local behavior of the Fₙ near a point, which would typically look like tendsto_uniformly_on_filter F f p (𝓝 x). Still, while this may be the "correct" definition (see tendsto_uniformly_on_iff_tendsto_uniformly_on_filter), it is somewhat unwieldy to work with in practice. Thus, we provide the more traditional definition in tendsto_uniformly_on.

Most results hold under weaker assumptions of locally uniform approximation. In a first section, we prove the results under these weaker assumptions. Then, we derive the results on uniform convergence from them.

Tags #

Uniform limit, uniform convergence, tends uniformly to

Different notions of uniform convergence #

We define uniform convergence and locally uniform convergence, on a set or in the whole space.

def tendsto_uniformly_on_filter {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] (F : ι α β) (f : α β) (p : filter ι) (p' : filter α) :
Prop

A sequence of functions Fₙ converges uniformly on a filter p' to a limiting function f with respect to the filter p if, for any entourage of the diagonal u, one has p ×ᶠ p'-eventually (f x, Fₙ x) ∈ u.

Equations
theorem tendsto_uniformly_on_filter_iff_tendsto {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {p : filter ι} {p' : filter α} :
tendsto_uniformly_on_filter F f p p' filter.tendsto (λ (q : ι × α), (f q.snd, F q.fst q.snd)) (p.prod p') (uniformity β)

A sequence of functions Fₙ converges uniformly on a filter p' to a limiting function f w.r.t. filter p iff the function (n, x) ↦ (f x, Fₙ x) converges along p ×ᶠ p' to the uniformity. In other words: one knows nothing about the behavior of x in this limit besides it being in p'.

def tendsto_uniformly_on {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] (F : ι α β) (f : α β) (p : filter ι) (s : set α) :
Prop

A sequence of functions Fₙ converges uniformly on a set s to a limiting function f with respect to the filter p if, for any entourage of the diagonal u, one has p-eventually (f x, Fₙ x) ∈ u for all x ∈ s.

Equations
theorem tendsto_uniformly_on_iff_tendsto_uniformly_on_filter {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {s : set α} {p : filter ι} :
theorem tendsto_uniformly_on_filter.tendsto_uniformly_on {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {s : set α} {p : filter ι} :

Alias of the reverse direction of tendsto_uniformly_on_iff_tendsto_uniformly_on_filter.

theorem tendsto_uniformly_on.tendsto_uniformly_on_filter {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {s : set α} {p : filter ι} :

Alias of the forward direction of tendsto_uniformly_on_iff_tendsto_uniformly_on_filter.

theorem tendsto_uniformly_on_iff_tendsto {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {p : filter ι} {s : set α} :
tendsto_uniformly_on F f p s filter.tendsto (λ (q : ι × α), (f q.snd, F q.fst q.snd)) (p.prod (filter.principal s)) (uniformity β)

A sequence of functions Fₙ converges uniformly on a set s to a limiting function f w.r.t. filter p iff the function (n, x) ↦ (f x, Fₙ x) converges along p ×ᶠ 𝓟 s to the uniformity. In other words: one knows nothing about the behavior of x in this limit besides it being in s.

def tendsto_uniformly {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] (F : ι α β) (f : α β) (p : filter ι) :
Prop

A sequence of functions Fₙ converges uniformly to a limiting function f with respect to a filter p if, for any entourage of the diagonal u, one has p-eventually (f x, Fₙ x) ∈ u for all x.

Equations
theorem tendsto_uniformly_iff_tendsto_uniformly_on_filter {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {p : filter ι} :
theorem tendsto_uniformly.tendsto_uniformly_on_filter {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {p : filter ι} (h : tendsto_uniformly F f p) :
theorem tendsto_uniformly_on_iff_tendsto_uniformly_comp_coe {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {s : set α} {p : filter ι} :
tendsto_uniformly_on F f p s tendsto_uniformly (λ (i : ι) (x : s), F i x) (f coe) p
theorem tendsto_uniformly_iff_tendsto {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {p : filter ι} :
tendsto_uniformly F f p filter.tendsto (λ (q : ι × α), (f q.snd, F q.fst q.snd)) (p.prod ) (uniformity β)

A sequence of functions Fₙ converges uniformly to a limiting function f w.r.t. filter p iff the function (n, x) ↦ (f x, Fₙ x) converges along p ×ᶠ ⊤ to the uniformity. In other words: one knows nothing about the behavior of x in this limit.

theorem tendsto_uniformly_on_filter.tendsto_at {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {x : α} {p : filter ι} {p' : filter α} (h : tendsto_uniformly_on_filter F f p p') (hx : filter.principal {x} p') :
filter.tendsto (λ (n : ι), F n x) p (nhds (f x))

Uniform converence implies pointwise convergence.

theorem tendsto_uniformly_on.tendsto_at {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {s : set α} {p : filter ι} (h : tendsto_uniformly_on F f p s) {x : α} (hx : x s) :
filter.tendsto (λ (n : ι), F n x) p (nhds (f x))

Uniform converence implies pointwise convergence.

theorem tendsto_uniformly.tendsto_at {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {p : filter ι} (h : tendsto_uniformly F f p) (x : α) :
filter.tendsto (λ (n : ι), F n x) p (nhds (f x))

Uniform converence implies pointwise convergence.

theorem tendsto_uniformly_on_univ {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {p : filter ι} :
theorem tendsto_uniformly_on_filter.mono_left {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {p : filter ι} {p' : filter α} {p'' : filter ι} (h : tendsto_uniformly_on_filter F f p p') (hp : p'' p) :
theorem tendsto_uniformly_on_filter.mono_right {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {p : filter ι} {p' p'' : filter α} (h : tendsto_uniformly_on_filter F f p p') (hp : p'' p') :
theorem tendsto_uniformly_on.mono {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {s : set α} {p : filter ι} {s' : set α} (h : tendsto_uniformly_on F f p s) (h' : s' s) :
theorem tendsto_uniformly_on_filter.congr {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {p : filter ι} {p' : filter α} {F' : ι α β} (hf : tendsto_uniformly_on_filter F f p p') (hff' : ∀ᶠ (n : ι × α) in p.prod p', F n.fst n.snd = F' n.fst n.snd) :
theorem tendsto_uniformly_on.congr {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {s : set α} {p : filter ι} {F' : ι α β} (hf : tendsto_uniformly_on F f p s) (hff' : ∀ᶠ (n : ι) in p, set.eq_on (F n) (F' n) s) :
theorem tendsto_uniformly_on.congr_right {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {s : set α} {p : filter ι} {g : α β} (hf : tendsto_uniformly_on F f p s) (hfg : set.eq_on f g s) :
@[protected]
theorem tendsto_uniformly.tendsto_uniformly_on {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {s : set α} {p : filter ι} (h : tendsto_uniformly F f p) :
theorem tendsto_uniformly_on_filter.comp {α : Type u_1} {β : Type u_2} {γ : Type u_3} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {p : filter ι} {p' : filter α} (h : tendsto_uniformly_on_filter F f p p') (g : γ α) :
tendsto_uniformly_on_filter (λ (n : ι), F n g) (f g) p (filter.comap g p')

Composing on the right by a function preserves uniform convergence on a filter

theorem tendsto_uniformly_on.comp {α : Type u_1} {β : Type u_2} {γ : Type u_3} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {s : set α} {p : filter ι} (h : tendsto_uniformly_on F f p s) (g : γ α) :
tendsto_uniformly_on (λ (n : ι), F n g) (f g) p (g ⁻¹' s)

Composing on the right by a function preserves uniform convergence on a set

theorem tendsto_uniformly.comp {α : Type u_1} {β : Type u_2} {γ : Type u_3} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {p : filter ι} (h : tendsto_uniformly F f p) (g : γ α) :
tendsto_uniformly (λ (n : ι), F n g) (f g) p

Composing on the right by a function preserves uniform convergence

theorem uniform_continuous.comp_tendsto_uniformly_on_filter {α : Type u_1} {β : Type u_2} {γ : Type u_3} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {p : filter ι} {p' : filter α} [uniform_space γ] {g : β γ} (hg : uniform_continuous g) (h : tendsto_uniformly_on_filter F f p p') :
tendsto_uniformly_on_filter (λ (i : ι), g F i) (g f) p p'

Composing on the left by a uniformly continuous function preserves uniform convergence on a filter

theorem uniform_continuous.comp_tendsto_uniformly_on {α : Type u_1} {β : Type u_2} {γ : Type u_3} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {s : set α} {p : filter ι} [uniform_space γ] {g : β γ} (hg : uniform_continuous g) (h : tendsto_uniformly_on F f p s) :
tendsto_uniformly_on (λ (i : ι), g F i) (g f) p s

Composing on the left by a uniformly continuous function preserves uniform convergence on a set

theorem uniform_continuous.comp_tendsto_uniformly {α : Type u_1} {β : Type u_2} {γ : Type u_3} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {p : filter ι} [uniform_space γ] {g : β γ} (hg : uniform_continuous g) (h : tendsto_uniformly F f p) :
tendsto_uniformly (λ (i : ι), g F i) (g f) p

Composing on the left by a uniformly continuous function preserves uniform convergence

theorem tendsto_uniformly_on_filter.prod_map {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {p : filter ι} {p' : filter α} {ι' : Type u_3} {α' : Type u_5} {β' : Type u_6} [uniform_space β'] {F' : ι' α' β'} {f' : α' β'} {q : filter ι'} {q' : filter α'} (h : tendsto_uniformly_on_filter F f p p') (h' : tendsto_uniformly_on_filter F' f' q q') :
tendsto_uniformly_on_filter (λ (i : ι × ι'), prod.map (F i.fst) (F' i.snd)) (prod.map f f') (p.prod q) (p'.prod q')
theorem tendsto_uniformly_on.prod_map {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {s : set α} {p : filter ι} {ι' : Type u_3} {α' : Type u_5} {β' : Type u_6} [uniform_space β'] {F' : ι' α' β'} {f' : α' β'} {p' : filter ι'} {s' : set α'} (h : tendsto_uniformly_on F f p s) (h' : tendsto_uniformly_on F' f' p' s') :
tendsto_uniformly_on (λ (i : ι × ι'), prod.map (F i.fst) (F' i.snd)) (prod.map f f') (p.prod p') (s ×ˢ s')
theorem tendsto_uniformly.prod_map {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {p : filter ι} {ι' : Type u_3} {α' : Type u_5} {β' : Type u_6} [uniform_space β'] {F' : ι' α' β'} {f' : α' β'} {p' : filter ι'} (h : tendsto_uniformly F f p) (h' : tendsto_uniformly F' f' p') :
tendsto_uniformly (λ (i : ι × ι'), prod.map (F i.fst) (F' i.snd)) (prod.map f f') (p.prod p')
theorem tendsto_uniformly_on_filter.prod {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {p : filter ι} {p' : filter α} {ι' : Type u_3} {β' : Type u_5} [uniform_space β'] {F' : ι' α β'} {f' : α β'} {q : filter ι'} (h : tendsto_uniformly_on_filter F f p p') (h' : tendsto_uniformly_on_filter F' f' q p') :
tendsto_uniformly_on_filter (λ (i : ι × ι') (a : α), (F i.fst a, F' i.snd a)) (λ (a : α), (f a, f' a)) (p.prod q) p'
theorem tendsto_uniformly_on.prod {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {s : set α} {p : filter ι} {ι' : Type u_3} {β' : Type u_5} [uniform_space β'] {F' : ι' α β'} {f' : α β'} {p' : filter ι'} (h : tendsto_uniformly_on F f p s) (h' : tendsto_uniformly_on F' f' p' s) :
tendsto_uniformly_on (λ (i : ι × ι') (a : α), (F i.fst a, F' i.snd a)) (λ (a : α), (f a, f' a)) (p.prod p') s
theorem tendsto_uniformly.prod {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {p : filter ι} {ι' : Type u_3} {β' : Type u_5} [uniform_space β'] {F' : ι' α β'} {f' : α β'} {p' : filter ι'} (h : tendsto_uniformly F f p) (h' : tendsto_uniformly F' f' p') :
tendsto_uniformly (λ (i : ι × ι') (a : α), (F i.fst a, F' i.snd a)) (λ (a : α), (f a, f' a)) (p.prod p')
theorem tendsto_prod_filter_iff {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {p : filter ι} {p' : filter α} {c : β} :
filter.tendsto F (p.prod p') (nhds c) tendsto_uniformly_on_filter F (λ (_x : α), c) p p'

Uniform convergence on a filter p' to a constant function is equivalent to convergence in p ×ᶠ p'.

theorem tendsto_prod_principal_iff {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {s : set α} {p : filter ι} {c : β} :
filter.tendsto F (p.prod (filter.principal s)) (nhds c) tendsto_uniformly_on F (λ (_x : α), c) p s

Uniform convergence on a set s to a constant function is equivalent to convergence in p ×ᶠ 𝓟 s.

theorem tendsto_prod_top_iff {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {p : filter ι} {c : β} :
filter.tendsto F (p.prod ) (nhds c) tendsto_uniformly F (λ (_x : α), c) p

Uniform convergence to a constant function is equivalent to convergence in p ×ᶠ ⊤.

theorem tendsto_uniformly_on_empty {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {p : filter ι} :

Uniform convergence on the empty set is vacuously true

theorem tendsto_uniformly_on_singleton_iff_tendsto {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {x : α} {p : filter ι} :
tendsto_uniformly_on F f p {x} filter.tendsto (λ (n : ι), F n x) p (nhds (f x))

Uniform convergence on a singleton is equivalent to regular convergence

theorem filter.tendsto.tendsto_uniformly_on_filter_const {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {p : filter ι} {g : ι β} {b : β} (hg : filter.tendsto g p (nhds b)) (p' : filter α) :
tendsto_uniformly_on_filter (λ (n : ι) (a : α), g n) (λ (a : α), b) p p'

If a sequence g converges to some b, then the sequence of constant functions λ n, λ a, g n converges to the constant function λ a, b on any set s

theorem filter.tendsto.tendsto_uniformly_on_const {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {p : filter ι} {g : ι β} {b : β} (hg : filter.tendsto g p (nhds b)) (s : set α) :
tendsto_uniformly_on (λ (n : ι) (a : α), g n) (λ (a : α), b) p s

If a sequence g converges to some b, then the sequence of constant functions λ n, λ a, g n converges to the constant function λ a, b on any set s

theorem uniform_continuous_on.tendsto_uniformly {α : Type u_1} {β : Type u_2} {γ : Type u_3} [uniform_space β] [uniform_space α] [uniform_space γ] {x : α} {U : set α} (hU : U nhds x) {F : α β γ} (hF : uniform_continuous_on F (U ×ˢ set.univ)) :
theorem uniform_continuous₂.tendsto_uniformly {α : Type u_1} {β : Type u_2} {γ : Type u_3} [uniform_space β] [uniform_space α] [uniform_space γ] {f : α β γ} (h : uniform_continuous₂ f) {x : α} :
def uniform_cauchy_seq_on_filter {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] (F : ι α β) (p : filter ι) (p' : filter α) :
Prop

A sequence is uniformly Cauchy if eventually all of its pairwise differences are uniformly bounded

Equations
def uniform_cauchy_seq_on {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] (F : ι α β) (p : filter ι) (s : set α) :
Prop

A sequence is uniformly Cauchy if eventually all of its pairwise differences are uniformly bounded

Equations
theorem uniform_cauchy_seq_on.uniform_cauchy_seq_on_filter {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {s : set α} {p : filter ι} (hF : uniform_cauchy_seq_on F p s) :
theorem tendsto_uniformly_on_filter.uniform_cauchy_seq_on_filter {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {p : filter ι} {p' : filter α} (hF : tendsto_uniformly_on_filter F f p p') :

A sequence that converges uniformly is also uniformly Cauchy

theorem tendsto_uniformly_on.uniform_cauchy_seq_on {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {s : set α} {p : filter ι} (hF : tendsto_uniformly_on F f p s) :

A sequence that converges uniformly is also uniformly Cauchy

theorem uniform_cauchy_seq_on_filter.tendsto_uniformly_on_filter_of_tendsto {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {p : filter ι} {p' : filter α} [p.ne_bot] (hF : uniform_cauchy_seq_on_filter F p p') (hF' : ∀ᶠ (x : α) in p', filter.tendsto (λ (n : ι), F n x) p (nhds (f x))) :

A uniformly Cauchy sequence converges uniformly to its limit

theorem uniform_cauchy_seq_on.tendsto_uniformly_on_of_tendsto {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {s : set α} {p : filter ι} [p.ne_bot] (hF : uniform_cauchy_seq_on F p s) (hF' : (x : α), x s filter.tendsto (λ (n : ι), F n x) p (nhds (f x))) :

A uniformly Cauchy sequence converges uniformly to its limit

theorem uniform_cauchy_seq_on_filter.mono_left {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {p : filter ι} {p' : filter α} {p'' : filter ι} (hf : uniform_cauchy_seq_on_filter F p p') (hp : p'' p) :
theorem uniform_cauchy_seq_on_filter.mono_right {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {p : filter ι} {p' p'' : filter α} (hf : uniform_cauchy_seq_on_filter F p p') (hp : p'' p') :
theorem uniform_cauchy_seq_on.mono {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {s : set α} {p : filter ι} {s' : set α} (hf : uniform_cauchy_seq_on F p s) (hss' : s' s) :
theorem uniform_cauchy_seq_on_filter.comp {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {p : filter ι} {p' : filter α} {γ : Type u_3} (hf : uniform_cauchy_seq_on_filter F p p') (g : γ α) :
uniform_cauchy_seq_on_filter (λ (n : ι), F n g) p (filter.comap g p')

Composing on the right by a function preserves uniform Cauchy sequences

theorem uniform_cauchy_seq_on.comp {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {s : set α} {p : filter ι} {γ : Type u_3} (hf : uniform_cauchy_seq_on F p s) (g : γ α) :
uniform_cauchy_seq_on (λ (n : ι), F n g) p (g ⁻¹' s)

Composing on the right by a function preserves uniform Cauchy sequences

theorem uniform_continuous.comp_uniform_cauchy_seq_on {α : Type u_1} {β : Type u_2} {γ : Type u_3} {ι : Type u_4} [uniform_space β] {F : ι α β} {s : set α} {p : filter ι} [uniform_space γ] {g : β γ} (hg : uniform_continuous g) (hf : uniform_cauchy_seq_on F p s) :
uniform_cauchy_seq_on (λ (n : ι), g F n) p s

Composing on the left by a uniformly continuous function preserves uniform Cauchy sequences

theorem uniform_cauchy_seq_on.prod_map {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {s : set α} {p : filter ι} {ι' : Type u_3} {α' : Type u_5} {β' : Type u_6} [uniform_space β'] {F' : ι' α' β'} {p' : filter ι'} {s' : set α'} (h : uniform_cauchy_seq_on F p s) (h' : uniform_cauchy_seq_on F' p' s') :
uniform_cauchy_seq_on (λ (i : ι × ι'), prod.map (F i.fst) (F' i.snd)) (p.prod p') (s ×ˢ s')
theorem uniform_cauchy_seq_on.prod {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {s : set α} {p : filter ι} {ι' : Type u_3} {β' : Type u_5} [uniform_space β'] {F' : ι' α β'} {p' : filter ι'} (h : uniform_cauchy_seq_on F p s) (h' : uniform_cauchy_seq_on F' p' s) :
uniform_cauchy_seq_on (λ (i : ι × ι') (a : α), (F i.fst a, F' i.snd a)) (p.prod p') s
theorem uniform_cauchy_seq_on.prod' {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {s : set α} {p : filter ι} {β' : Type u_3} [uniform_space β'] {F' : ι α β'} (h : uniform_cauchy_seq_on F p s) (h' : uniform_cauchy_seq_on F' p s) :
uniform_cauchy_seq_on (λ (i : ι) (a : α), (F i a, F' i a)) p s
theorem uniform_cauchy_seq_on.cauchy_map {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {s : set α} {x : α} {p : filter ι} [hp : p.ne_bot] (hf : uniform_cauchy_seq_on F p s) (hx : x s) :
cauchy (filter.map (λ (i : ι), F i x) p)

If a sequence of functions is uniformly Cauchy on a set, then the values at each point form a Cauchy sequence.

theorem tendsto_uniformly_on_of_seq_tendsto_uniformly_on {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {s : set α} {l : filter ι} [l.is_countably_generated] (h : (u : ι), filter.tendsto u filter.at_top l tendsto_uniformly_on (λ (n : ), F (u n)) f filter.at_top s) :
theorem tendsto_uniformly_on.seq_tendsto_uniformly_on {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {s : set α} {l : filter ι} (h : tendsto_uniformly_on F f l s) (u : ι) (hu : filter.tendsto u filter.at_top l) :
tendsto_uniformly_on (λ (n : ), F (u n)) f filter.at_top s
theorem tendsto_uniformly_on_iff_seq_tendsto_uniformly_on {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {s : set α} {l : filter ι} [l.is_countably_generated] :
theorem tendsto_uniformly_iff_seq_tendsto_uniformly {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {l : filter ι} [l.is_countably_generated] :
def tendsto_locally_uniformly_on {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] [topological_space α] (F : ι α β) (f : α β) (p : filter ι) (s : set α) :
Prop

A sequence of functions Fₙ converges locally uniformly on a set s to a limiting function f with respect to a filter p if, for any entourage of the diagonal u, for any x ∈ s, one has p-eventually (f y, Fₙ y) ∈ u for all y in a neighborhood of x in s.

Equations
def tendsto_locally_uniformly {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] [topological_space α] (F : ι α β) (f : α β) (p : filter ι) :
Prop

A sequence of functions Fₙ converges locally uniformly to a limiting function f with respect to a filter p if, for any entourage of the diagonal u, for any x, one has p-eventually (f y, Fₙ y) ∈ u for all y in a neighborhood of x.

Equations
theorem tendsto_locally_uniformly_on_iff_tendsto_locally_uniformly_comp_coe {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {s : set α} {p : filter ι} [topological_space α] :
tendsto_locally_uniformly_on F f p s tendsto_locally_uniformly (λ (i : ι) (x : s), F i x) (f coe) p
theorem tendsto_locally_uniformly_iff_forall_tendsto {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {p : filter ι} [topological_space α] :
tendsto_locally_uniformly F f p (x : α), filter.tendsto (λ (y : ι × α), (f y.snd, F y.fst y.snd)) (p.prod (nhds x)) (uniformity β)
@[protected]
theorem tendsto_uniformly_on.tendsto_locally_uniformly_on {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {s : set α} {p : filter ι} [topological_space α] (h : tendsto_uniformly_on F f p s) :
@[protected]
theorem tendsto_uniformly.tendsto_locally_uniformly {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {p : filter ι} [topological_space α] (h : tendsto_uniformly F f p) :
theorem tendsto_locally_uniformly_on.mono {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {s s' : set α} {p : filter ι} [topological_space α] (h : tendsto_locally_uniformly_on F f p s) (h' : s' s) :
theorem tendsto_locally_uniformly_on_Union {α : Type u_1} {β : Type u_2} {γ : Type u_3} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {p : filter ι} [topological_space α] {S : γ set α} (hS : (i : γ), is_open (S i)) (h : (i : γ), tendsto_locally_uniformly_on F f p (S i)) :
tendsto_locally_uniformly_on F f p ( (i : γ), S i)
theorem tendsto_locally_uniformly_on_bUnion {α : Type u_1} {β : Type u_2} {γ : Type u_3} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {p : filter ι} [topological_space α] {s : set γ} {S : γ set α} (hS : (i : γ), i s is_open (S i)) (h : (i : γ), i s tendsto_locally_uniformly_on F f p (S i)) :
tendsto_locally_uniformly_on F f p ( (i : γ) (H : i s), S i)
theorem tendsto_locally_uniformly_on_sUnion {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {p : filter ι} [topological_space α] (S : set (set α)) (hS : (s : set α), s S is_open s) (h : (s : set α), s S tendsto_locally_uniformly_on F f p s) :
theorem tendsto_locally_uniformly_on.union {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {p : filter ι} [topological_space α] {s₁ s₂ : set α} (hs₁ : is_open s₁) (hs₂ : is_open s₂) (h₁ : tendsto_locally_uniformly_on F f p s₁) (h₂ : tendsto_locally_uniformly_on F f p s₂) :
theorem tendsto_locally_uniformly_on_univ {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {p : filter ι} [topological_space α] :
@[protected]
theorem tendsto_locally_uniformly.tendsto_locally_uniformly_on {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {s : set α} {p : filter ι} [topological_space α] (h : tendsto_locally_uniformly F f p) :
theorem tendsto_locally_uniformly_iff_tendsto_uniformly_of_compact_space {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {p : filter ι} [topological_space α] [compact_space α] :

On a compact space, locally uniform convergence is just uniform convergence.

theorem tendsto_locally_uniformly_on_iff_tendsto_uniformly_on_of_compact {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {s : set α} {p : filter ι} [topological_space α] (hs : is_compact s) :

For a compact set s, locally uniform convergence on s is just uniform convergence on s.

theorem tendsto_locally_uniformly_on.comp {α : Type u_1} {β : Type u_2} {γ : Type u_3} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {s : set α} {p : filter ι} [topological_space α] [topological_space γ] {t : set γ} (h : tendsto_locally_uniformly_on F f p s) (g : γ α) (hg : set.maps_to g t s) (cg : continuous_on g t) :
tendsto_locally_uniformly_on (λ (n : ι), F n g) (f g) p t
theorem tendsto_locally_uniformly.comp {α : Type u_1} {β : Type u_2} {γ : Type u_3} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {p : filter ι} [topological_space α] [topological_space γ] (h : tendsto_locally_uniformly F f p) (g : γ α) (cg : continuous g) :
tendsto_locally_uniformly (λ (n : ι), F n g) (f g) p
theorem tendsto_locally_uniformly_on_tfae {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {s : set α} [topological_space α] [locally_compact_space α] (G : ι α β) (g : α β) (p : filter ι) (hs : is_open s) :
[tendsto_locally_uniformly_on G g p s, (K : set α), K s is_compact K tendsto_uniformly_on G g p K, (x : α), x s ( (v : set α) (H : v nhds_within x s), tendsto_uniformly_on G g p v)].tfae
theorem tendsto_locally_uniformly_on_iff_forall_is_compact {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {s : set α} {p : filter ι} [topological_space α] [locally_compact_space α] (hs : is_open s) :
theorem tendsto_locally_uniformly_on_iff_filter {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {s : set α} {p : filter ι} [topological_space α] :
theorem tendsto_locally_uniformly_iff_filter {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {p : filter ι} [topological_space α] :
theorem tendsto_locally_uniformly_on.tendsto_at {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {s : set α} {p : filter ι} [topological_space α] (hf : tendsto_locally_uniformly_on F f p s) {a : α} (ha : a s) :
filter.tendsto (λ (i : ι), F i a) p (nhds (f a))
theorem tendsto_locally_uniformly_on.unique {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {s : set α} {p : filter ι} [topological_space α] [p.ne_bot] [t2_space β] {g : α β} (hf : tendsto_locally_uniformly_on F f p s) (hg : tendsto_locally_uniformly_on F g p s) :
set.eq_on f g s
theorem tendsto_locally_uniformly_on.congr {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {s : set α} {p : filter ι} [topological_space α] {G : ι α β} (hf : tendsto_locally_uniformly_on F f p s) (hg : (n : ι), set.eq_on (F n) (G n) s) :
theorem tendsto_locally_uniformly_on.congr_right {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {s : set α} {p : filter ι} [topological_space α] {g : α β} (hf : tendsto_locally_uniformly_on F f p s) (hg : set.eq_on f g s) :

Uniform approximation #

In this section, we give lemmas ensuring that a function is continuous if it can be approximated uniformly by continuous functions. We give various versions, within a set or the whole space, at a single point or at all points, with locally uniform approximation or uniform approximation. All the statements are derived from a statement about locally uniform approximation within a set at a point, called continuous_within_at_of_locally_uniform_approx_of_continuous_within_at.

theorem continuous_within_at_of_locally_uniform_approx_of_continuous_within_at {α : Type u_1} {β : Type u_2} [uniform_space β] {f : α β} {s : set α} {x : α} [topological_space α] (hx : x s) (L : (u : set × β)), u uniformity β ( (t : set α) (H : t nhds_within x s) (F : α β), continuous_within_at F s x (y : α), y t (f y, F y) u)) :

A function which can be locally uniformly approximated by functions which are continuous within a set at a point is continuous within this set at this point.

theorem continuous_at_of_locally_uniform_approx_of_continuous_at {α : Type u_1} {β : Type u_2} [uniform_space β] {f : α β} {x : α} [topological_space α] (L : (u : set × β)), u uniformity β ( (t : set α) (H : t nhds x) (F : α β), continuous_at F x (y : α), y t (f y, F y) u)) :

A function which can be locally uniformly approximated by functions which are continuous at a point is continuous at this point.

theorem continuous_on_of_locally_uniform_approx_of_continuous_within_at {α : Type u_1} {β : Type u_2} [uniform_space β] {f : α β} {s : set α} [topological_space α] (L : (x : α), x s (u : set × β)), u uniformity β ( (t : set α) (H : t nhds_within x s) (F : α β), continuous_within_at F s x (y : α), y t (f y, F y) u)) :

A function which can be locally uniformly approximated by functions which are continuous on a set is continuous on this set.

theorem continuous_on_of_uniform_approx_of_continuous_on {α : Type u_1} {β : Type u_2} [uniform_space β] {f : α β} {s : set α} [topological_space α] (L : (u : set × β)), u uniformity β ( (F : α β), continuous_on F s (y : α), y s (f y, F y) u)) :

A function which can be uniformly approximated by functions which are continuous on a set is continuous on this set.

theorem continuous_of_locally_uniform_approx_of_continuous_at {α : Type u_1} {β : Type u_2} [uniform_space β] {f : α β} [topological_space α] (L : (x : α) (u : set × β)), u uniformity β ( (t : set α) (H : t nhds x) (F : α β), continuous_at F x (y : α), y t (f y, F y) u)) :

A function which can be locally uniformly approximated by continuous functions is continuous.

theorem continuous_of_uniform_approx_of_continuous {α : Type u_1} {β : Type u_2} [uniform_space β] {f : α β} [topological_space α] (L : (u : set × β)), u uniformity β ( (F : α β), continuous F (y : α), (f y, F y) u)) :

A function which can be uniformly approximated by continuous functions is continuous.

Uniform limits #

From the previous statements on uniform approximation, we deduce continuity results for uniform limits.

@[protected]
theorem tendsto_locally_uniformly_on.continuous_on {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {s : set α} {p : filter ι} [topological_space α] (h : tendsto_locally_uniformly_on F f p s) (hc : ∀ᶠ (n : ι) in p, continuous_on (F n) s) [p.ne_bot] :

A locally uniform limit on a set of functions which are continuous on this set is itself continuous on this set.

@[protected]
theorem tendsto_uniformly_on.continuous_on {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {s : set α} {p : filter ι} [topological_space α] (h : tendsto_uniformly_on F f p s) (hc : ∀ᶠ (n : ι) in p, continuous_on (F n) s) [p.ne_bot] :

A uniform limit on a set of functions which are continuous on this set is itself continuous on this set.

@[protected]
theorem tendsto_locally_uniformly.continuous {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {p : filter ι} [topological_space α] (h : tendsto_locally_uniformly F f p) (hc : ∀ᶠ (n : ι) in p, continuous (F n)) [p.ne_bot] :

A locally uniform limit of continuous functions is continuous.

@[protected]
theorem tendsto_uniformly.continuous {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {p : filter ι} [topological_space α] (h : tendsto_uniformly F f p) (hc : ∀ᶠ (n : ι) in p, continuous (F n)) [p.ne_bot] :

A uniform limit of continuous functions is continuous.

Composing limits under uniform convergence #

In general, if Fₙ converges pointwise to a function f, and gₙ tends to x, it is not true that Fₙ gₙ tends to f x. It is true however if the convergence of Fₙ to f is uniform. In this paragraph, we prove variations around this statement.

theorem tendsto_comp_of_locally_uniform_limit_within {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {s : set α} {x : α} {p : filter ι} {g : ι α} [topological_space α] (h : continuous_within_at f s x) (hg : filter.tendsto g p (nhds_within x s)) (hunif : (u : set × β)), u uniformity β ( (t : set α) (H : t nhds_within x s), ∀ᶠ (n : ι) in p, (y : α), y t (f y, F n y) u)) :
filter.tendsto (λ (n : ι), F n (g n)) p (nhds (f x))

If Fₙ converges locally uniformly on a neighborhood of x within a set s to a function f which is continuous at x within s, and gₙ tends to x within s, then Fₙ (gₙ) tends to f x.

theorem tendsto_comp_of_locally_uniform_limit {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {x : α} {p : filter ι} {g : ι α} [topological_space α] (h : continuous_at f x) (hg : filter.tendsto g p (nhds x)) (hunif : (u : set × β)), u uniformity β ( (t : set α) (H : t nhds x), ∀ᶠ (n : ι) in p, (y : α), y t (f y, F n y) u)) :
filter.tendsto (λ (n : ι), F n (g n)) p (nhds (f x))

If Fₙ converges locally uniformly on a neighborhood of x to a function f which is continuous at x, and gₙ tends to x, then Fₙ (gₙ) tends to f x.

theorem tendsto_locally_uniformly_on.tendsto_comp {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {s : set α} {x : α} {p : filter ι} {g : ι α} [topological_space α] (h : tendsto_locally_uniformly_on F f p s) (hf : continuous_within_at f s x) (hx : x s) (hg : filter.tendsto g p (nhds_within x s)) :
filter.tendsto (λ (n : ι), F n (g n)) p (nhds (f x))

If Fₙ tends locally uniformly to f on a set s, and gₙ tends to x within s, then Fₙ gₙ tends to f x if f is continuous at x within s and x ∈ s.

theorem tendsto_uniformly_on.tendsto_comp {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {s : set α} {x : α} {p : filter ι} {g : ι α} [topological_space α] (h : tendsto_uniformly_on F f p s) (hf : continuous_within_at f s x) (hg : filter.tendsto g p (nhds_within x s)) :
filter.tendsto (λ (n : ι), F n (g n)) p (nhds (f x))

If Fₙ tends uniformly to f on a set s, and gₙ tends to x within s, then Fₙ gₙ tends to f x if f is continuous at x within s.

theorem tendsto_locally_uniformly.tendsto_comp {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {x : α} {p : filter ι} {g : ι α} [topological_space α] (h : tendsto_locally_uniformly F f p) (hf : continuous_at f x) (hg : filter.tendsto g p (nhds x)) :
filter.tendsto (λ (n : ι), F n (g n)) p (nhds (f x))

If Fₙ tends locally uniformly to f, and gₙ tends to x, then Fₙ gₙ tends to f x.

theorem tendsto_uniformly.tendsto_comp {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι α β} {f : α β} {x : α} {p : filter ι} {g : ι α} [topological_space α] (h : tendsto_uniformly F f p) (hf : continuous_at f x) (hg : filter.tendsto g p (nhds x)) :
filter.tendsto (λ (n : ι), F n (g n)) p (nhds (f x))

If Fₙ tends uniformly to f, and gₙ tends to x, then Fₙ gₙ tends to f x.