mathlib documentation

topology.uniform_space.uniform_convergence

Uniform convergence #

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.

Implementation notes #

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 {α : 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 {α : 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 ×ᶠ 𝓟 s) (𝓤 β)

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_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 ×ᶠ ) (𝓤 β)

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.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 (𝓝 (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.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) :
@[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.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 tendsto_uniformly_on.comp' {α : Type u_1} {β : Type u_2} {γ : Type u_3} {ι : Type u_4} [uniform_space β] {F : ι → α → β} {f : α → β} {s : set α} {p : filter ι} [uniform_space γ] {g : β → γ} (h : tendsto_uniformly_on F f p s) (hg : uniform_continuous g) :
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 tendsto_uniformly.comp' {α : Type u_1} {β : Type u_2} {γ : Type u_3} {ι : Type u_4} [uniform_space β] {F : ι → α → β} {f : α → β} {p : filter ι} [uniform_space γ] {g : β → γ} (h : tendsto_uniformly F f p) (hg : uniform_continuous g) :
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.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 ×ᶠ 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 ×ᶠ 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 ×ᶠ 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 ×ᶠ p')
theorem tendsto_prod_top_iff {α : Type u_1} {β : Type u_2} {ι : Type u_4} [uniform_space β] {F : ι → α → β} {p : filter ι} {c : β} :
filter.tendsto F (p ×ᶠ ) (𝓝 c) tendsto_uniformly F (λ (_x : α), c) p

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

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 𝓝 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 : α} :
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 ltendsto_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] :
tendsto_uniformly_on F f l s ∀ (u : → ι), filter.tendsto u filter.at_top ltendsto_uniformly_on (λ (n : ), F (u n)) f filter.at_top s
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] :
tendsto_uniformly F f l ∀ (u : → ι), filter.tendsto u filter.at_top ltendsto_uniformly (λ (n : ), F (u n)) f filter.at_top
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 ×ᶠ 𝓝 x) (𝓤 β)
@[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_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

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 𝓤 β(∃ (t : set α) (H : t 𝓝[s] x) (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 𝓤 β(∃ (t : set α) (H : t 𝓝 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 𝓤 β(∃ (t : set α) (H : t 𝓝[s] x) (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 𝓤 β(∃ (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 𝓤 β(∃ (t : set α) (H : t 𝓝 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 𝓤 β(∃ (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 (𝓝[s] x)) (hunif : ∀ (u : set × β)), u 𝓤 β(∃ (t : set α) (H : t 𝓝[s] x), ∀ᶠ (n : ι) in p, ∀ (y : α), y t(f y, F n y) u)) :
filter.tendsto (λ (n : ι), F n (g n)) p (𝓝 (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 (𝓝 x)) (hunif : ∀ (u : set × β)), u 𝓤 β(∃ (t : set α) (H : t 𝓝 x), ∀ᶠ (n : ι) in p, ∀ (y : α), y t(f y, F n y) u)) :
filter.tendsto (λ (n : ι), F n (g n)) p (𝓝 (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 (𝓝[s] x)) :
filter.tendsto (λ (n : ι), F n (g n)) p (𝓝 (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 (𝓝[s] x)) :
filter.tendsto (λ (n : ι), F n (g n)) p (𝓝 (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 (𝓝 x)) :
filter.tendsto (λ (n : ι), F n (g n)) p (𝓝 (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 (𝓝 x)) :
filter.tendsto (λ (n : ι), F n (g n)) p (𝓝 (f x))

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