Documentation

Mathlib.Analysis.Analytic.Within

Properties of analyticity restricted to a set #

From Mathlib.Analysis.Analytic.Basic, we have the definitions

  1. AnalyticWithinAt ๐•œ f s x means a power series at x converges to f on ๐“[s] x, and f is continuous within s at x.
  2. AnalyticWithinOn ๐•œ f s t means โˆ€ x โˆˆ t, AnalyticWithinAt ๐•œ f s x.

This means there exists an extension of f which is analytic and agrees with f on s โˆช {x}, but f is allowed to be arbitrary elsewhere. Requiring ContinuousWithinAt is essential if x โˆ‰ s: it is required for composition and smoothness to follow without extra hypotheses (we could alternately require convergence at x even if x โˆ‰ s).

Here we prove basic properties of these definitions. Where convenient we assume completeness of the ambient space, which allows us to related AnalyticWithinAt to analyticity of a local extension.

Basic properties #

@[simp]
theorem hasFPowerSeriesWithinOnBall_univ {๐•œ : Type u_1} [NontriviallyNormedField ๐•œ] {E : Type u_2} {F : Type u_3} [NormedAddCommGroup E] [NormedSpace ๐•œ E] [NormedAddCommGroup F] [NormedSpace ๐•œ F] {f : E โ†’ F} {p : FormalMultilinearSeries ๐•œ E F} {x : E} {r : ENNReal} :
@[simp]
theorem hasFPowerSeriesWithinAt_univ {๐•œ : Type u_1} [NontriviallyNormedField ๐•œ] {E : Type u_2} {F : Type u_3} [NormedAddCommGroup E] [NormedSpace ๐•œ E] [NormedAddCommGroup F] [NormedSpace ๐•œ F] {f : E โ†’ F} {p : FormalMultilinearSeries ๐•œ E F} {x : E} :
@[simp]
theorem analyticWithinAt_univ {๐•œ : Type u_1} [NontriviallyNormedField ๐•œ] {E : Type u_2} {F : Type u_3} [NormedAddCommGroup E] [NormedSpace ๐•œ E] [NormedAddCommGroup F] [NormedSpace ๐•œ F] {f : E โ†’ F} {x : E} :
AnalyticWithinAt ๐•œ f Set.univ x โ†” AnalyticAt ๐•œ f x
theorem analyticWithinOn_univ {๐•œ : Type u_1} [NontriviallyNormedField ๐•œ] {E : Type u_2} {F : Type u_3} [NormedAddCommGroup E] [NormedSpace ๐•œ E] [NormedAddCommGroup F] [NormedSpace ๐•œ F] {f : E โ†’ F} :
AnalyticWithinOn ๐•œ f Set.univ โ†” AnalyticOn ๐•œ f Set.univ
theorem HasFPowerSeriesWithinAt.continuousWithinAt {๐•œ : Type u_1} [NontriviallyNormedField ๐•œ] {E : Type u_2} {F : Type u_3} [NormedAddCommGroup E] [NormedSpace ๐•œ E] [NormedAddCommGroup F] [NormedSpace ๐•œ F] {f : E โ†’ F} {p : FormalMultilinearSeries ๐•œ E F} {s : Set E} {x : E} (h : HasFPowerSeriesWithinAt f p s x) :
theorem AnalyticWithinAt.continuousWithinAt {๐•œ : Type u_1} [NontriviallyNormedField ๐•œ] {E : Type u_2} {F : Type u_3} [NormedAddCommGroup E] [NormedSpace ๐•œ E] [NormedAddCommGroup F] [NormedSpace ๐•œ F] {f : E โ†’ F} {s : Set E} {x : E} (h : AnalyticWithinAt ๐•œ f s x) :
theorem analyticWithinAt_of_singleton_mem {๐•œ : Type u_1} [NontriviallyNormedField ๐•œ] {E : Type u_2} {F : Type u_3} [NormedAddCommGroup E] [NormedSpace ๐•œ E] [NormedAddCommGroup F] [NormedSpace ๐•œ F] {f : E โ†’ F} {s : Set E} {x : E} (h : {x} โˆˆ nhdsWithin x s) :
AnalyticWithinAt ๐•œ f s x

AnalyticWithinAt is trivial if {x} โˆˆ ๐“[s] x

theorem AnalyticAt.analyticWithinAt {๐•œ : Type u_1} [NontriviallyNormedField ๐•œ] {E : Type u_2} {F : Type u_3} [NormedAddCommGroup E] [NormedSpace ๐•œ E] [NormedAddCommGroup F] [NormedSpace ๐•œ F] {f : E โ†’ F} {s : Set E} {x : E} (h : AnalyticAt ๐•œ f x) :
AnalyticWithinAt ๐•œ f s x

Analyticity implies analyticity within any s

theorem AnalyticOn.analyticWithinOn {๐•œ : Type u_1} [NontriviallyNormedField ๐•œ] {E : Type u_2} {F : Type u_3} [NormedAddCommGroup E] [NormedSpace ๐•œ E] [NormedAddCommGroup F] [NormedSpace ๐•œ F] {f : E โ†’ F} {s : Set E} (h : AnalyticOn ๐•œ f s) :
AnalyticWithinOn ๐•œ f s

Analyticity on s implies analyticity within s

theorem AnalyticWithinOn.continuousOn {๐•œ : Type u_1} [NontriviallyNormedField ๐•œ] {E : Type u_2} {F : Type u_3} [NormedAddCommGroup E] [NormedSpace ๐•œ E] [NormedAddCommGroup F] [NormedSpace ๐•œ F] {f : E โ†’ F} {s : Set E} (h : AnalyticWithinOn ๐•œ f s) :
theorem analyticWithinOn_of_locally_analyticWithinOn {๐•œ : Type u_1} [NontriviallyNormedField ๐•œ] {E : Type u_2} {F : Type u_3} [NormedAddCommGroup E] [NormedSpace ๐•œ E] [NormedAddCommGroup F] [NormedSpace ๐•œ F] {f : E โ†’ F} {s : Set E} (h : โˆ€ x โˆˆ s, โˆƒ (u : Set E), IsOpen u โˆง x โˆˆ u โˆง AnalyticWithinOn ๐•œ f (s โˆฉ u)) :
AnalyticWithinOn ๐•œ f s

If f is AnalyticWithinOn near each point in a set, it is AnalyticWithinOn the set

@[simp]
theorem IsOpen.analyticWithinOn_iff_analyticOn {๐•œ : Type u_1} [NontriviallyNormedField ๐•œ] {E : Type u_2} {F : Type u_3} [NormedAddCommGroup E] [NormedSpace ๐•œ E] [NormedAddCommGroup F] [NormedSpace ๐•œ F] {f : E โ†’ F} {s : Set E} (hs : IsOpen s) :
AnalyticWithinOn ๐•œ f s โ†” AnalyticOn ๐•œ f s

On open sets, AnalyticOn and AnalyticWithinOn coincide

Equivalence to analyticity of a local extension #

We show that HasFPowerSeriesWithinOnBall, HasFPowerSeriesWithinAt, and AnalyticWithinAt are equivalent to the existence of a local extension with full analyticity. We do not yet show a result for AnalyticWithinOn, as this requires a bit more work to show that local extensions can be stitched together.

theorem hasFPowerSeriesWithinOnBall_iff_exists_hasFPowerSeriesOnBall {๐•œ : Type u_1} [NontriviallyNormedField ๐•œ] {E : Type u_2} {F : Type u_3} [NormedAddCommGroup E] [NormedSpace ๐•œ E] [NormedAddCommGroup F] [NormedSpace ๐•œ F] [CompleteSpace F] {f : E โ†’ F} {p : FormalMultilinearSeries ๐•œ E F} {s : Set E} {x : E} {r : ENNReal} :

f has power series p at x iff some local extension of f has that series

theorem hasFPowerSeriesWithinAt_iff_exists_hasFPowerSeriesAt {๐•œ : Type u_1} [NontriviallyNormedField ๐•œ] {E : Type u_2} {F : Type u_3} [NormedAddCommGroup E] [NormedSpace ๐•œ E] [NormedAddCommGroup F] [NormedSpace ๐•œ F] [CompleteSpace F] {f : E โ†’ F} {p : FormalMultilinearSeries ๐•œ E F} {s : Set E} {x : E} :

f has power series p at x iff some local extension of f has that series

theorem analyticWithinAt_iff_exists_analyticAt {๐•œ : Type u_1} [NontriviallyNormedField ๐•œ] {E : Type u_2} {F : Type u_3} [NormedAddCommGroup E] [NormedSpace ๐•œ E] [NormedAddCommGroup F] [NormedSpace ๐•œ F] [CompleteSpace F] {f : E โ†’ F} {s : Set E} {x : E} :
AnalyticWithinAt ๐•œ f s x โ†” ContinuousWithinAt f s x โˆง โˆƒ (g : E โ†’ F), f =แถ [nhdsWithin x s] g โˆง AnalyticAt ๐•œ g x

f is analytic within s at x iff some local extension of f is analytic at x

theorem AnalyticWithinAt.exists_analyticAt {๐•œ : Type u_1} [NontriviallyNormedField ๐•œ] {E : Type u_2} {F : Type u_3} [NormedAddCommGroup E] [NormedSpace ๐•œ E] [NormedAddCommGroup F] [NormedSpace ๐•œ F] [CompleteSpace F] {f : E โ†’ F} {s : Set E} {x : E} (h : AnalyticWithinAt ๐•œ f s x) :
โˆƒ (g : E โ†’ F), f x = g x โˆง f =แถ [nhdsWithin x s] g โˆง AnalyticAt ๐•œ g x

If f is analytic within s at x, some local extension of f is analytic at x

Congruence #

We require completeness to use equivalence to locally extensions, but this is nonessential.

theorem AnalyticWithinAt.congr_of_eventuallyEq {๐•œ : Type u_1} [NontriviallyNormedField ๐•œ] {E : Type u_2} {F : Type u_3} [NormedAddCommGroup E] [NormedSpace ๐•œ E] [NormedAddCommGroup F] [NormedSpace ๐•œ F] [CompleteSpace F] {f : E โ†’ F} {g : E โ†’ F} {s : Set E} {x : E} (hf : AnalyticWithinAt ๐•œ f s x) (hs : f =แถ [nhdsWithin x s] g) (hx : f x = g x) :
AnalyticWithinAt ๐•œ g s x
theorem AnalyticWithinAt.congr {๐•œ : Type u_1} [NontriviallyNormedField ๐•œ] {E : Type u_2} {F : Type u_3} [NormedAddCommGroup E] [NormedSpace ๐•œ E] [NormedAddCommGroup F] [NormedSpace ๐•œ F] [CompleteSpace F] {f : E โ†’ F} {g : E โ†’ F} {s : Set E} {x : E} (hf : AnalyticWithinAt ๐•œ f s x) (hs : Set.EqOn f g s) (hx : f x = g x) :
AnalyticWithinAt ๐•œ g s x
theorem AnalyticWithinOn.congr {๐•œ : Type u_1} [NontriviallyNormedField ๐•œ] {E : Type u_2} {F : Type u_3} [NormedAddCommGroup E] [NormedSpace ๐•œ E] [NormedAddCommGroup F] [NormedSpace ๐•œ F] [CompleteSpace F] {f : E โ†’ F} {g : E โ†’ F} {s : Set E} (hf : AnalyticWithinOn ๐•œ f s) (hs : Set.EqOn f g s) :
AnalyticWithinOn ๐•œ g s

Monotonicity w.r.t. the set we're analytic within #

theorem HasFPowerSeriesWithinOnBall.mono {๐•œ : Type u_1} [NontriviallyNormedField ๐•œ] {E : Type u_2} {F : Type u_3} [NormedAddCommGroup E] [NormedSpace ๐•œ E] [NormedAddCommGroup F] [NormedSpace ๐•œ F] {f : E โ†’ F} {p : FormalMultilinearSeries ๐•œ E F} {s : Set E} {t : Set E} {x : E} {r : ENNReal} (h : HasFPowerSeriesWithinOnBall f p t x r) (hs : s โŠ† t) :
theorem HasFPowerSeriesWithinAt.mono {๐•œ : Type u_1} [NontriviallyNormedField ๐•œ] {E : Type u_2} {F : Type u_3} [NormedAddCommGroup E] [NormedSpace ๐•œ E] [NormedAddCommGroup F] [NormedSpace ๐•œ F] {f : E โ†’ F} {p : FormalMultilinearSeries ๐•œ E F} {s : Set E} {t : Set E} {x : E} (h : HasFPowerSeriesWithinAt f p t x) (hs : s โŠ† t) :
theorem AnalyticWithinAt.mono {๐•œ : Type u_1} [NontriviallyNormedField ๐•œ] {E : Type u_2} {F : Type u_3} [NormedAddCommGroup E] [NormedSpace ๐•œ E] [NormedAddCommGroup F] [NormedSpace ๐•œ F] {f : E โ†’ F} {s : Set E} {t : Set E} {x : E} (h : AnalyticWithinAt ๐•œ f t x) (hs : s โŠ† t) :
AnalyticWithinAt ๐•œ f s x
theorem AnalyticWithinOn.mono {๐•œ : Type u_1} [NontriviallyNormedField ๐•œ] {E : Type u_2} {F : Type u_3} [NormedAddCommGroup E] [NormedSpace ๐•œ E] [NormedAddCommGroup F] [NormedSpace ๐•œ F] {f : E โ†’ F} {s : Set E} {t : Set E} (h : AnalyticWithinOn ๐•œ f t) (hs : s โŠ† t) :
AnalyticWithinOn ๐•œ f s

Analyticity within respects composition #

Currently we require CompleteSpaces to use equivalence to local extensions, but this is not essential.

theorem AnalyticWithinAt.comp {๐•œ : Type u_1} [NontriviallyNormedField ๐•œ] {E : Type u_2} {F : Type u_3} {G : Type u_4} [NormedAddCommGroup E] [NormedSpace ๐•œ E] [NormedAddCommGroup F] [NormedSpace ๐•œ F] [NormedAddCommGroup G] [NormedSpace ๐•œ G] [CompleteSpace F] [CompleteSpace G] {f : F โ†’ G} {g : E โ†’ F} {s : Set F} {t : Set E} {x : E} (hf : AnalyticWithinAt ๐•œ f s (g x)) (hg : AnalyticWithinAt ๐•œ g t x) (h : Set.MapsTo g t s) :
AnalyticWithinAt ๐•œ (f โˆ˜ g) t x
theorem AnalyticWithinOn.comp {๐•œ : Type u_1} [NontriviallyNormedField ๐•œ] {E : Type u_2} {F : Type u_3} {G : Type u_4} [NormedAddCommGroup E] [NormedSpace ๐•œ E] [NormedAddCommGroup F] [NormedSpace ๐•œ F] [NormedAddCommGroup G] [NormedSpace ๐•œ G] [CompleteSpace F] [CompleteSpace G] {f : F โ†’ G} {g : E โ†’ F} {s : Set F} {t : Set E} (hf : AnalyticWithinOn ๐•œ f s) (hg : AnalyticWithinOn ๐•œ g t) (h : Set.MapsTo g t s) :
AnalyticWithinOn ๐•œ (f โˆ˜ g) t

Analyticity within implies smoothness #

theorem AnalyticWithinAt.contDiffWithinAt {๐•œ : Type u_1} [NontriviallyNormedField ๐•œ] {E : Type u_2} {F : Type u_3} [NormedAddCommGroup E] [NormedSpace ๐•œ E] [NormedAddCommGroup F] [NormedSpace ๐•œ F] [CompleteSpace F] {f : E โ†’ F} {s : Set E} {x : E} (h : AnalyticWithinAt ๐•œ f s x) {n : โ„•โˆž} :
ContDiffWithinAt ๐•œ n f s x
theorem AnalyticWithinOn.contDiffOn {๐•œ : Type u_1} [NontriviallyNormedField ๐•œ] {E : Type u_2} {F : Type u_3} [NormedAddCommGroup E] [NormedSpace ๐•œ E] [NormedAddCommGroup F] [NormedSpace ๐•œ F] [CompleteSpace F] {f : E โ†’ F} {s : Set E} (h : AnalyticWithinOn ๐•œ f s) {n : โ„•โˆž} :
ContDiffOn ๐•œ n f s

Analyticity within respects products #

theorem HasFPowerSeriesWithinOnBall.prod {๐•œ : Type u_1} [NontriviallyNormedField ๐•œ] {E : Type u_2} {F : Type u_3} {G : Type u_4} [NormedAddCommGroup E] [NormedSpace ๐•œ E] [NormedAddCommGroup F] [NormedSpace ๐•œ F] [NormedAddCommGroup G] [NormedSpace ๐•œ G] {e : E} {f : E โ†’ F} {g : E โ†’ G} {s : Set E} {r : ENNReal} {t : ENNReal} {p : FormalMultilinearSeries ๐•œ E F} {q : FormalMultilinearSeries ๐•œ E G} (hf : HasFPowerSeriesWithinOnBall f p s e r) (hg : HasFPowerSeriesWithinOnBall g q s e t) :
HasFPowerSeriesWithinOnBall (fun (x : E) => (f x, g x)) (p.prod q) s e (min r t)
theorem HasFPowerSeriesWithinAt.prod {๐•œ : Type u_1} [NontriviallyNormedField ๐•œ] {E : Type u_2} {F : Type u_3} {G : Type u_4} [NormedAddCommGroup E] [NormedSpace ๐•œ E] [NormedAddCommGroup F] [NormedSpace ๐•œ F] [NormedAddCommGroup G] [NormedSpace ๐•œ G] {e : E} {f : E โ†’ F} {g : E โ†’ G} {s : Set E} {p : FormalMultilinearSeries ๐•œ E F} {q : FormalMultilinearSeries ๐•œ E G} (hf : HasFPowerSeriesWithinAt f p s e) (hg : HasFPowerSeriesWithinAt g q s e) :
HasFPowerSeriesWithinAt (fun (x : E) => (f x, g x)) (p.prod q) s e
theorem AnalyticWithinAt.prod {๐•œ : Type u_1} [NontriviallyNormedField ๐•œ] {E : Type u_2} {F : Type u_3} {G : Type u_4} [NormedAddCommGroup E] [NormedSpace ๐•œ E] [NormedAddCommGroup F] [NormedSpace ๐•œ F] [NormedAddCommGroup G] [NormedSpace ๐•œ G] {e : E} {f : E โ†’ F} {g : E โ†’ G} {s : Set E} (hf : AnalyticWithinAt ๐•œ f s e) (hg : AnalyticWithinAt ๐•œ g s e) :
AnalyticWithinAt ๐•œ (fun (x : E) => (f x, g x)) s e
theorem AnalyticWithinOn.prod {๐•œ : Type u_1} [NontriviallyNormedField ๐•œ] {E : Type u_2} {F : Type u_3} {G : Type u_4} [NormedAddCommGroup E] [NormedSpace ๐•œ E] [NormedAddCommGroup F] [NormedSpace ๐•œ F] [NormedAddCommGroup G] [NormedSpace ๐•œ G] {f : E โ†’ F} {g : E โ†’ G} {s : Set E} (hf : AnalyticWithinOn ๐•œ f s) (hg : AnalyticWithinOn ๐•œ g s) :
AnalyticWithinOn ๐•œ (fun (x : E) => (f x, g x)) s