Documentation

Mathlib.Analysis.CStarAlgebra.ContinuousFunctionalCalculus.Continuity

Continuity of the continuous functional calculus in each variable #

The continuous functional calculus is a map which takes a pair a : A (A is a C⋆-algebra) and a function f : C(spectrum R a, R) where a satisfies some predicate p, depending on R and returns another element of the algebra A. This is the map cfcHom. The class ContinuousFunctionalCalculus declares that cfcHom is a continuous map from C(spectrum R a, R) to A. However, users generally interact with the continuous functional calculus through cfc, which operates on bare functions f : R → R instead and takes a junk value when f is not continuous on the spectrum of a. In this file we provide some lemma concerning the continuity of cfc, subject to natural hypotheses.

However, the continuous functional calculus is also continuous in the variable a, but there are some conditions that must be satisfied. In particular, given a function f : R → R the map a ↦ cfc f a is continuous so long as a varies over a collection of elements satisfying the predicate p and their spectra are collectively contained in a compact set on which f is continuous. Moreover, it is required that the continuous functional calculus be the isometric variant.

Finally, all of this is developed for both the unital and non-unital functional calculi. The continuity results in the function variable are valid for all scalar rings, but the continuity results in the variable a come in two flavors: those for RCLike 𝕜 and those for ℝ≥0.

To do #

theorem tendsto_cfc_fun {X : Type u_1} {R : Type u_2} {A : Type u_3} {p : AProp} [CommSemiring R] [StarRing R] [MetricSpace R] [IsTopologicalSemiring R] [ContinuousStar R] [Ring A] [StarRing A] [TopologicalSpace A] [Algebra R A] [ContinuousFunctionalCalculus R A p] {l : Filter X} {F : XRR} {f : RR} {a : A} (h_tendsto : TendstoUniformlyOn F f l (spectrum R a)) (hF : ∀ᶠ (x : X) in l, ContinuousOn (F x) (spectrum R a)) :
Filter.Tendsto (fun (x : X) => cfc (F x) a) l (nhds (cfc f a))

If F : X → R → R tends to f : R → R uniformly on the spectrum of a, and all these functions are continuous on the spectrum, then fun x ↦ cfc (F x) a tends to cfc f a.

theorem continuousAt_cfc_fun {X : Type u_1} {R : Type u_2} {A : Type u_3} {p : AProp} [CommSemiring R] [StarRing R] [MetricSpace R] [IsTopologicalSemiring R] [ContinuousStar R] [Ring A] [StarRing A] [TopologicalSpace A] [Algebra R A] [ContinuousFunctionalCalculus R A p] [TopologicalSpace X] {f : XRR} {a : A} {x₀ : X} (h_tendsto : TendstoUniformlyOn f (f x₀) (nhds x₀) (spectrum R a)) (hf : ∀ᶠ (x : X) in nhds x₀, ContinuousOn (f x) (spectrum R a)) :
ContinuousAt (fun (x : X) => cfc (f x) a) x₀

If f : X → R → R tends to f x₀ uniformly (along 𝓝 x₀) on the spectrum of a, and each f x is continuous on the spectrum of a, then fun x ↦ cfc (f x) a is continuous at x₀.

theorem continuousWithinAt_cfc_fun {X : Type u_1} {R : Type u_2} {A : Type u_3} {p : AProp} [CommSemiring R] [StarRing R] [MetricSpace R] [IsTopologicalSemiring R] [ContinuousStar R] [Ring A] [StarRing A] [TopologicalSpace A] [Algebra R A] [ContinuousFunctionalCalculus R A p] [TopologicalSpace X] {f : XRR} {a : A} {x₀ : X} {s : Set X} (h_tendsto : TendstoUniformlyOn f (f x₀) (nhdsWithin x₀ s) (spectrum R a)) (hf : ∀ᶠ (x : X) in nhdsWithin x₀ s, ContinuousOn (f x) (spectrum R a)) :
ContinuousWithinAt (fun (x : X) => cfc (f x) a) s x₀

If f : X → R → R tends to f x₀ uniformly (along 𝓝[s] x₀) on the spectrum of a, and eventually each f x is continuous on the spectrum of a, then fun x ↦ cfc (f x) a is continuous at x₀ within s.

theorem ContinuousOn.cfc_fun {X : Type u_1} {R : Type u_2} {A : Type u_3} {p : AProp} [CommSemiring R] [StarRing R] [MetricSpace R] [IsTopologicalSemiring R] [ContinuousStar R] [Ring A] [StarRing A] [TopologicalSpace A] [Algebra R A] [ContinuousFunctionalCalculus R A p] [TopologicalSpace X] {f : XRR} {a : A} {s : Set X} (h_cont : ContinuousOn (fun (x : X) => (UniformOnFun.ofFun {spectrum R a}) (f x)) s) (hf : xs, ContinuousOn (f x) (spectrum R a) := by cfc_cont_tac) :
ContinuousOn (fun (x : X) => cfc (f x) a) s

If f : X → R → R is continuous on s : Set X in the topology on X → R →ᵤ[{spectrum R a}] → R, and each f is continuous on the spectrum, then x ↦ cfc (f x) a is continuous on s also.

theorem Continuous.cfc_fun {X : Type u_1} {R : Type u_2} {A : Type u_3} {p : AProp} [CommSemiring R] [StarRing R] [MetricSpace R] [IsTopologicalSemiring R] [ContinuousStar R] [Ring A] [StarRing A] [TopologicalSpace A] [Algebra R A] [ContinuousFunctionalCalculus R A p] [TopologicalSpace X] (f : XRR) (a : A) (h_cont : Continuous fun (x : X) => (UniformOnFun.ofFun {spectrum R a}) (f x)) (hf : ∀ (x : X), ContinuousOn (f x) (spectrum R a) := by cfc_cont_tac) :
Continuous fun (x : X) => cfc (f x) a

If f : X → R → R is continuous in the topology on X → R →ᵤ[{spectrum R a}] → R, and each f is continuous on the spectrum, then x ↦ cfc (f x) a is continuous.

theorem continuous_cfcHomSuperset_left {X : Type u_1} {𝕜 : Type u_2} {A : Type u_3} {p : AProp} [RCLike 𝕜] [NormedRing A] [StarRing A] [NormedAlgebra 𝕜 A] [IsometricContinuousFunctionalCalculus 𝕜 A p] [ContinuousStar A] [TopologicalSpace X] {s : Set 𝕜} (hs : IsCompact s) (f : C(s, 𝕜)) (a : XA) (ha_cont : Continuous a) (ha : ∀ (x : X), spectrum 𝕜 (a x) s) (ha' : ∀ (x : X), p (a x) := by cfc_tac) :
Continuous fun (x : X) => (cfcHomSuperset ) f

cfcHomSuperset is continuous in the variable a : A when s : Set 𝕜 is compact and a varies over elements whose spectrum is contained in s, all of which satisfy the predicate p.

theorem continuousOn_cfc {𝕜 : Type u_2} (A : Type u_3) {p : AProp} [RCLike 𝕜] [NormedRing A] [StarRing A] [NormedAlgebra 𝕜 A] [IsometricContinuousFunctionalCalculus 𝕜 A p] [ContinuousStar A] {s : Set 𝕜} (hs : IsCompact s) (f : 𝕜𝕜) (hf : ContinuousOn f s := by cfc_cont_tac) :
ContinuousOn (cfc f) {a : A | p a spectrum 𝕜 a s}

For f : 𝕜 → 𝕜 continuous on a compact set s, cfc f is continuous on the set of a : A satisfying the predicate p (associated to 𝕜) and whose 𝕜-spectrum is contained in s.

theorem Filter.Tendsto.cfc {X : Type u_1} {𝕜 : Type u_2} {A : Type u_3} {p : AProp} [RCLike 𝕜] [NormedRing A] [StarRing A] [NormedAlgebra 𝕜 A] [IsometricContinuousFunctionalCalculus 𝕜 A p] [ContinuousStar A] {s : Set 𝕜} (hs : IsCompact s) (f : 𝕜𝕜) {a : XA} {a₀ : A} {l : Filter X} (ha_tendsto : Tendsto a l (nhds a₀)) (ha : ∀ᶠ (x : X) in l, spectrum 𝕜 (a x) s) (ha' : ∀ᶠ (x : X) in l, p (a x)) (ha₀ : spectrum 𝕜 a₀ s) (ha₀' : p a₀) (hf : ContinuousOn f s := by cfc_cont_tac) :
Tendsto (fun (x : X) => cfc f (a x)) l (nhds (cfc f a₀))

If f : 𝕜 → 𝕜 is continuous on a compact set s and a : X → A tends to a₀ : A along a filter l (such that eventually a x satisfies the predicate p associated to 𝕜 and has spectrum contained in s, as does a₀), then fun x ↦ cfc f (a x) tends to cfc f a₀.

theorem ContinuousAt.cfc {X : Type u_1} {𝕜 : Type u_2} {A : Type u_3} {p : AProp} [RCLike 𝕜] [NormedRing A] [StarRing A] [NormedAlgebra 𝕜 A] [IsometricContinuousFunctionalCalculus 𝕜 A p] [ContinuousStar A] [TopologicalSpace X] {s : Set 𝕜} (hs : IsCompact s) (f : 𝕜𝕜) {a : XA} {x₀ : X} (ha_cont : ContinuousAt a x₀) (ha : ∀ᶠ (x : X) in nhds x₀, spectrum 𝕜 (a x) s) (ha' : ∀ᶠ (x : X) in nhds x₀, p (a x)) (hf : ContinuousOn f s := by cfc_cont_tac) :
ContinuousAt (fun (x : X) => cfc f (a x)) x₀

If f : 𝕜 → 𝕜 is continuous on a compact set s and a : X → A is continuous at x₀, and eventually a x satisfies the predicate p associated to 𝕜 and has spectrum contained in s), then fun x ↦ cfc f (a x) is continuous at x₀.

theorem ContinuousWithinAt.cfc {X : Type u_1} {𝕜 : Type u_2} {A : Type u_3} {p : AProp} [RCLike 𝕜] [NormedRing A] [StarRing A] [NormedAlgebra 𝕜 A] [IsometricContinuousFunctionalCalculus 𝕜 A p] [ContinuousStar A] [TopologicalSpace X] {s : Set 𝕜} (hs : IsCompact s) (f : 𝕜𝕜) {a : XA} {x₀ : X} {t : Set X} (hx₀ : x₀ t) (ha_cont : ContinuousWithinAt a t x₀) (ha : ∀ᶠ (x : X) in nhdsWithin x₀ t, spectrum 𝕜 (a x) s) (ha' : ∀ᶠ (x : X) in nhdsWithin x₀ t, p (a x)) (hf : ContinuousOn f s := by cfc_cont_tac) :
ContinuousWithinAt (fun (x : X) => cfc f (a x)) t x₀

If f : 𝕜 → 𝕜 is continuous on a compact set s and a : X → A is continuous at x₀ within a set t : Set X, and eventually a x satisfies the predicate p associated to 𝕜 and has spectrum contained in s), then fun x ↦ cfc f (a x) is continuous at x₀ within t.

theorem ContinuousOn.cfc {X : Type u_1} {𝕜 : Type u_2} {A : Type u_3} {p : AProp} [RCLike 𝕜] [NormedRing A] [StarRing A] [NormedAlgebra 𝕜 A] [IsometricContinuousFunctionalCalculus 𝕜 A p] [ContinuousStar A] [TopologicalSpace X] {s : Set 𝕜} (hs : IsCompact s) (f : 𝕜𝕜) {a : XA} {t : Set X} (ha_cont : ContinuousOn a t) (ha : xt, spectrum 𝕜 (a x) s) (ha' : xt, p (a x)) (hf : ContinuousOn f s := by cfc_cont_tac) :
ContinuousOn (fun (x : X) => cfc f (a x)) t

If f : 𝕜 → 𝕜 is continuous on a compact set s and a : X → A is continuous on t : Set X, and a x satisfies the predicate p associated to 𝕜 and has spectrum contained in s for all x ∈ t, then fun x ↦ cfc f (a x) is continuous on t.

theorem Continuous.cfc {X : Type u_1} {𝕜 : Type u_2} {A : Type u_3} {p : AProp} [RCLike 𝕜] [NormedRing A] [StarRing A] [NormedAlgebra 𝕜 A] [IsometricContinuousFunctionalCalculus 𝕜 A p] [ContinuousStar A] [TopologicalSpace X] {s : Set 𝕜} (hs : IsCompact s) (f : 𝕜𝕜) {a : XA} (ha_cont : Continuous a) (ha : ∀ (x : X), spectrum 𝕜 (a x) s) (hf : ContinuousOn f s := by cfc_cont_tac) (ha' : ∀ (x : X), p (a x) := by cfc_tac) :
Continuous fun (x : X) => cfc f (a x)

cfc is continuous in the variable a : A when s : Set 𝕜 is compact and a varies over elements whose spectrum is contained in s, all of which satisfy the predicate p, and the function f is continuous on the spectrum of a.

theorem Filter.Tendsto.cfc_nnreal {X : Type u_1} {A : Type u_2} [NormedRing A] [StarRing A] [NormedAlgebra A] [IsometricContinuousFunctionalCalculus A IsSelfAdjoint] [ContinuousStar A] [PartialOrder A] [StarOrderedRing A] [NonnegSpectrumClass A] [T2Space A] [IsTopologicalRing A] {s : Set NNReal} (hs : IsCompact s) (f : NNRealNNReal) {a : XA} {a₀ : A} {l : Filter X} (ha_tendsto : Tendsto a l (nhds a₀)) (ha : ∀ᶠ (x : X) in l, spectrum NNReal (a x) s) (ha' : ∀ᶠ (x : X) in l, 0 a x) (ha₀ : spectrum NNReal a₀ s) (ha₀' : 0 a₀) (hf : ContinuousOn f s := by cfc_cont_tac) :
Tendsto (fun (x : X) => cfc f (a x)) l (nhds (cfc f a₀))

If f : ℝ≥0 → ℝ≥0 is continuous on a compact set s and a : X → A tends to a₀ : A along a filter l (such that eventually 0 ≤ a x and has spectrum contained in s, as does a₀), then fun x ↦ cfc f (a x) tends to cfc f a₀.

theorem ContinuousAt.cfc_nnreal {X : Type u_1} {A : Type u_2} [NormedRing A] [StarRing A] [NormedAlgebra A] [IsometricContinuousFunctionalCalculus A IsSelfAdjoint] [ContinuousStar A] [PartialOrder A] [StarOrderedRing A] [NonnegSpectrumClass A] [T2Space A] [IsTopologicalRing A] [TopologicalSpace X] {s : Set NNReal} (hs : IsCompact s) (f : NNRealNNReal) {a : XA} {x₀ : X} (ha_cont : ContinuousAt a x₀) (ha : ∀ᶠ (x : X) in nhds x₀, spectrum NNReal (a x) s) (ha' : ∀ᶠ (x : X) in nhds x₀, 0 a x) (hf : ContinuousOn f s := by cfc_cont_tac) :
ContinuousAt (fun (x : X) => cfc f (a x)) x₀

If f : ℝ≥0 → ℝ≥0 is continuous on a compact set s and a : X → A is continuous at x₀, and eventually 0 ≤ a x and has spectrum contained in s), then fun x ↦ cfc f (a x) is continuous at x₀.

theorem ContinuousWithinAt.cfc_nnreal {X : Type u_1} {A : Type u_2} [NormedRing A] [StarRing A] [NormedAlgebra A] [IsometricContinuousFunctionalCalculus A IsSelfAdjoint] [ContinuousStar A] [PartialOrder A] [StarOrderedRing A] [NonnegSpectrumClass A] [T2Space A] [IsTopologicalRing A] [TopologicalSpace X] {s : Set NNReal} (hs : IsCompact s) (f : NNRealNNReal) {a : XA} {x₀ : X} {t : Set X} (hx₀ : x₀ t) (ha_cont : ContinuousWithinAt a t x₀) (ha : ∀ᶠ (x : X) in nhdsWithin x₀ t, spectrum NNReal (a x) s) (ha' : ∀ᶠ (x : X) in nhdsWithin x₀ t, 0 a x) (hf : ContinuousOn f s := by cfc_cont_tac) :
ContinuousWithinAt (fun (x : X) => cfc f (a x)) t x₀

If f : ℝ≥0 → ℝ≥0 is continuous on a compact set s and a : X → A is continuous at x₀ within a set t : Set X, and eventually 0 ≤ a x and has spectrum contained in s), then fun x ↦ cfc f (a x) is continuous at x₀ within t.

theorem ContinuousOn.cfc_nnreal {X : Type u_1} {A : Type u_2} [NormedRing A] [StarRing A] [NormedAlgebra A] [IsometricContinuousFunctionalCalculus A IsSelfAdjoint] [ContinuousStar A] [PartialOrder A] [StarOrderedRing A] [NonnegSpectrumClass A] [T2Space A] [IsTopologicalRing A] [TopologicalSpace X] {s : Set NNReal} (hs : IsCompact s) (f : NNRealNNReal) {a : XA} {t : Set X} (ha_cont : ContinuousOn a t) (ha : xt, spectrum NNReal (a x) s) (ha' : xt, 0 a x) (hf : ContinuousOn f s := by cfc_cont_tac) :
ContinuousOn (fun (x : X) => cfc f (a x)) t

If f : ℝ≥0 → ℝ≥0 is continuous on a compact set s and a : X → A is continuous on t : Set X, and 0 ≤ a x and has spectrum contained in s for all x ∈ t, then fun x ↦ cfc f (a x) is continuous on t.

theorem Continuous.cfc_nnreal {X : Type u_1} {A : Type u_2} [NormedRing A] [StarRing A] [NormedAlgebra A] [IsometricContinuousFunctionalCalculus A IsSelfAdjoint] [ContinuousStar A] [PartialOrder A] [StarOrderedRing A] [NonnegSpectrumClass A] [T2Space A] [IsTopologicalRing A] [TopologicalSpace X] {s : Set NNReal} (hs : IsCompact s) (f : NNRealNNReal) {a : XA} (ha_cont : Continuous a) (ha : ∀ (x : X), spectrum NNReal (a x) s) (hf : ContinuousOn f s := by cfc_cont_tac) (ha' : ∀ (x : X), 0 a x := by cfc_tac) :
Continuous fun (x : X) => cfc f (a x)

cfc is continuous in the variable a : A when s : Set ℝ≥0 is compact and a varies over nonnegative elements whose spectrum is contained in s, and the function f is continuous on s.

theorem tendsto_cfcₙ_fun {X : Type u_1} {R : Type u_2} {A : Type u_3} {p : AProp} [CommSemiring R] [StarRing R] [MetricSpace R] [Nontrivial R] [IsTopologicalSemiring R] [ContinuousStar R] [NonUnitalRing A] [StarRing A] [TopologicalSpace A] [Module R A] [SMulCommClass R A A] [IsScalarTower R A A] [NonUnitalContinuousFunctionalCalculus R A p] {l : Filter X} {F : XRR} {f : RR} {a : A} (h_tendsto : TendstoUniformlyOn F f l (quasispectrum R a)) (hF : ∀ᶠ (x : X) in l, ContinuousOn (F x) (quasispectrum R a)) (hF0 : ∀ᶠ (x : X) in l, F x 0 = 0) :
Filter.Tendsto (fun (x : X) => cfcₙ (F x) a) l (nhds (cfcₙ f a))

If F : X → R → R tends to f : R → R uniformly on the spectrum of a, and all these functions are continuous on the spectrum and map zero to itself, then fun x ↦ cfcₙ (F x) a tends to cfcₙ f a.

theorem continuousAt_cfcₙ_fun {X : Type u_1} {R : Type u_2} {A : Type u_3} {p : AProp} [CommSemiring R] [StarRing R] [MetricSpace R] [Nontrivial R] [IsTopologicalSemiring R] [ContinuousStar R] [NonUnitalRing A] [StarRing A] [TopologicalSpace A] [Module R A] [SMulCommClass R A A] [IsScalarTower R A A] [NonUnitalContinuousFunctionalCalculus R A p] [TopologicalSpace X] {f : XRR} {a : A} {x₀ : X} (h_tendsto : TendstoUniformlyOn f (f x₀) (nhds x₀) (quasispectrum R a)) (hf : ∀ᶠ (x : X) in nhds x₀, ContinuousOn (f x) (quasispectrum R a)) (hf0 : ∀ᶠ (x : X) in nhds x₀, f x 0 = 0) :
ContinuousAt (fun (x : X) => cfcₙ (f x) a) x₀

If f : X → R → R tends to f x₀ uniformly (along 𝓝 x₀) on the spectrum of a, and each f x is continuous on the spectrum of a and maps zero to itself, then fun x ↦ cfcₙ (f x) a is continuous at x₀.

theorem continuousWithinAt_cfcₙ_fun {X : Type u_1} {R : Type u_2} {A : Type u_3} {p : AProp} [CommSemiring R] [StarRing R] [MetricSpace R] [Nontrivial R] [IsTopologicalSemiring R] [ContinuousStar R] [NonUnitalRing A] [StarRing A] [TopologicalSpace A] [Module R A] [SMulCommClass R A A] [IsScalarTower R A A] [NonUnitalContinuousFunctionalCalculus R A p] [TopologicalSpace X] {f : XRR} {a : A} {x₀ : X} {s : Set X} (h_tendsto : TendstoUniformlyOn f (f x₀) (nhdsWithin x₀ s) (quasispectrum R a)) (hf : ∀ᶠ (x : X) in nhdsWithin x₀ s, ContinuousOn (f x) (quasispectrum R a)) (hf0 : ∀ᶠ (x : X) in nhdsWithin x₀ s, f x 0 = 0 := by cfc_zero_tac) :
ContinuousWithinAt (fun (x : X) => cfcₙ (f x) a) s x₀

If f : X → R → R tends to f x₀ uniformly (along 𝓝[s] x₀) on the spectrum of a, and eventually each f x is continuous on the spectrum of a and maps zero to itself, then fun x ↦ cfcₙ (f x) a is continuous at x₀ within s.

theorem ContinuousOn.cfcₙ_fun {X : Type u_1} {R : Type u_2} {A : Type u_3} {p : AProp} [CommSemiring R] [StarRing R] [MetricSpace R] [Nontrivial R] [IsTopologicalSemiring R] [ContinuousStar R] [NonUnitalRing A] [StarRing A] [TopologicalSpace A] [Module R A] [SMulCommClass R A A] [IsScalarTower R A A] [NonUnitalContinuousFunctionalCalculus R A p] [TopologicalSpace X] {f : XRR} {a : A} {s : Set X} (h_cont : ContinuousOn (fun (x : X) => (UniformOnFun.ofFun {quasispectrum R a}) (f x)) s) (hf : xs, ContinuousOn (f x) (quasispectrum R a)) (hf0 : xs, f x 0 = 0) :
ContinuousOn (fun (x : X) => cfcₙ (f x) a) s

If f : X → R → R is continuous on s : Set X in the topology on X → R →ᵤ[{spectrum R a}] → R, and for each x ∈ s, f x is continuous on the spectrum and maps zero to itself, then x ↦ cfcₙ (f x) a is continuous on s also.

theorem Continuous.cfcₙ_fun {X : Type u_1} {R : Type u_2} {A : Type u_3} {p : AProp} [CommSemiring R] [StarRing R] [MetricSpace R] [Nontrivial R] [IsTopologicalSemiring R] [ContinuousStar R] [NonUnitalRing A] [StarRing A] [TopologicalSpace A] [Module R A] [SMulCommClass R A A] [IsScalarTower R A A] [NonUnitalContinuousFunctionalCalculus R A p] [TopologicalSpace X] (f : XRR) (a : A) (h_cont : Continuous fun (x : X) => (UniformOnFun.ofFun {quasispectrum R a}) (f x)) (hf : ∀ (x : X), ContinuousOn (f x) (quasispectrum R a) := by cfc_cont_tac) (hf0 : ∀ (x : X), f x 0 = 0 := by cfc_zero_tac) :
Continuous fun (x : X) => cfcₙ (f x) a

If f : X → R → R is continuous in the topology on X → R →ᵤ[{spectrum R a}] → R, and each f is continuous on the spectrum and maps zero to itself, then x ↦ cfcₙ (f x) a is continuous.

theorem continuous_cfcₙHomSuperset_left {X : Type u_1} {𝕜 : Type u_2} {A : Type u_3} {p : AProp} [RCLike 𝕜] [NonUnitalNormedRing A] [StarRing A] [NormedSpace 𝕜 A] [IsScalarTower 𝕜 A A] [SMulCommClass 𝕜 A A] [ContinuousStar A] [NonUnitalIsometricContinuousFunctionalCalculus 𝕜 A p] [TopologicalSpace X] {s : Set 𝕜} (hs : IsCompact s) [hs0 : Fact (0 s)] (f : ContinuousMapZero (↑s) 𝕜) {a : XA} (ha_cont : Continuous a) (ha : ∀ (x : X), quasispectrum 𝕜 (a x) s) (ha' : ∀ (x : X), p (a x) := by cfc_tac) :
Continuous fun (x : X) => (cfcₙHomSuperset ) f

cfcₙHomSuperset is continuous in the variable a : A when s : Set 𝕜 is compact and a varies over elements whose spectrum is contained in s, all of which satisfy the predicate p.

theorem continuousOn_cfcₙ {𝕜 : Type u_2} (A : Type u_3) {p : AProp} [RCLike 𝕜] [NonUnitalNormedRing A] [StarRing A] [NormedSpace 𝕜 A] [IsScalarTower 𝕜 A A] [SMulCommClass 𝕜 A A] [ContinuousStar A] [NonUnitalIsometricContinuousFunctionalCalculus 𝕜 A p] {s : Set 𝕜} (hs : IsCompact s) (f : 𝕜𝕜) (hf : ContinuousOn f s := by cfc_cont_tac) (hf0 : f 0 = 0 := by cfc_zero_tac) :
ContinuousOn (fun (x : A) => cfcₙ f x) {a : A | p a quasispectrum 𝕜 a s}

For f : 𝕜 → 𝕜 continuous on a set s for which f 0 = 0, cfcₙ f is continuous on the set of a : A satisfying the predicate p (associated to 𝕜) and whose 𝕜-quasispectrum is contained in s.

theorem Filter.Tendsto.cfcₙ {X : Type u_1} {𝕜 : Type u_2} {A : Type u_3} {p : AProp} [RCLike 𝕜] [NonUnitalNormedRing A] [StarRing A] [NormedSpace 𝕜 A] [IsScalarTower 𝕜 A A] [SMulCommClass 𝕜 A A] [ContinuousStar A] [NonUnitalIsometricContinuousFunctionalCalculus 𝕜 A p] {s : Set 𝕜} (hs : IsCompact s) (f : 𝕜𝕜) {a : XA} {a₀ : A} {l : Filter X} (ha_tendsto : Tendsto a l (nhds a₀)) (ha : ∀ᶠ (x : X) in l, quasispectrum 𝕜 (a x) s) (ha' : ∀ᶠ (x : X) in l, p (a x)) (ha₀ : quasispectrum 𝕜 a₀ s) (ha₀' : p a₀) (hf : ContinuousOn f s := by cfc_cont_tac) (hf0 : f 0 = 0 := by cfc_zero_tac) :
Tendsto (fun (x : X) => cfcₙ f (a x)) l (nhds (cfcₙ f a₀))

If f : 𝕜 → 𝕜 is continuous on a compact set s and f 0 = 0 and a : X → A tends to a₀ : A along a filter l (such that eventually a x satisfies the predicate p associated to 𝕜 and has quasispectrum contained in s, as does a₀), then fun x ↦ cfcₙ f (a x) tends to cfcₙ f a₀.

theorem ContinuousAt.cfcₙ {X : Type u_1} {𝕜 : Type u_2} {A : Type u_3} {p : AProp} [RCLike 𝕜] [NonUnitalNormedRing A] [StarRing A] [NormedSpace 𝕜 A] [IsScalarTower 𝕜 A A] [SMulCommClass 𝕜 A A] [ContinuousStar A] [NonUnitalIsometricContinuousFunctionalCalculus 𝕜 A p] [TopologicalSpace X] {s : Set 𝕜} (hs : IsCompact s) (f : 𝕜𝕜) {a : XA} {x₀ : X} (ha_cont : ContinuousAt a x₀) (ha : ∀ᶠ (x : X) in nhds x₀, quasispectrum 𝕜 (a x) s) (ha' : ∀ᶠ (x : X) in nhds x₀, p (a x)) (hf : ContinuousOn f s := by cfc_cont_tac) (hf0 : f 0 = 0 := by cfc_zero_tac) :
ContinuousAt (fun (x : X) => cfcₙ f (a x)) x₀

If f : 𝕜 → 𝕜 is continuous on a compact set s and f 0 = 0 and a : X → A is continuous at x₀, and eventually a x satisfies the predicate p associated to 𝕜 and has quasispectrum contained in s), then fun x ↦ cfcₙ f (a x) is continuous at x₀.

theorem ContinuousWithinAt.cfcₙ {X : Type u_1} {𝕜 : Type u_2} {A : Type u_3} {p : AProp} [RCLike 𝕜] [NonUnitalNormedRing A] [StarRing A] [NormedSpace 𝕜 A] [IsScalarTower 𝕜 A A] [SMulCommClass 𝕜 A A] [ContinuousStar A] [NonUnitalIsometricContinuousFunctionalCalculus 𝕜 A p] [TopologicalSpace X] {s : Set 𝕜} (hs : IsCompact s) (f : 𝕜𝕜) {a : XA} {x₀ : X} {t : Set X} (hx₀ : x₀ t) (ha_cont : ContinuousWithinAt a t x₀) (ha : ∀ᶠ (x : X) in nhdsWithin x₀ t, quasispectrum 𝕜 (a x) s) (ha' : ∀ᶠ (x : X) in nhdsWithin x₀ t, p (a x)) (hf : ContinuousOn f s := by cfc_cont_tac) (hf0 : f 0 = 0 := by cfc_zero_tac) :
ContinuousWithinAt (fun (x : X) => cfcₙ f (a x)) t x₀

If f : 𝕜 → 𝕜 is continuous on a compact set s and f 0 = 0 and a : X → A is continuous at x₀ within a set t : Set X, and eventually a x satisfies the predicate p associated to 𝕜 and has quasispectrum contained in s), then fun x ↦ cfcₙ f (a x) is continuous at x₀ within t.

theorem ContinuousOn.cfcₙ {X : Type u_1} {𝕜 : Type u_2} {A : Type u_3} {p : AProp} [RCLike 𝕜] [NonUnitalNormedRing A] [StarRing A] [NormedSpace 𝕜 A] [IsScalarTower 𝕜 A A] [SMulCommClass 𝕜 A A] [ContinuousStar A] [NonUnitalIsometricContinuousFunctionalCalculus 𝕜 A p] [TopologicalSpace X] {s : Set 𝕜} (hs : IsCompact s) (f : 𝕜𝕜) {a : XA} {t : Set X} (ha_cont : ContinuousOn a t) (ha : xt, quasispectrum 𝕜 (a x) s) (ha' : xt, p (a x)) (hf : ContinuousOn f s := by cfc_cont_tac) (hf0 : f 0 = 0 := by cfc_zero_tac) :
ContinuousOn (fun (x : X) => cfcₙ f (a x)) t

If f : 𝕜 → 𝕜 is continuous on a compact set s and f 0 = 0 and a : X → A is continuous on t : Set X, and a x satisfies the predicate p associated to 𝕜 and has quasispectrum contained in s for all x ∈ t, then fun x ↦ cfcₙ f (a x) is continuous on t.

theorem Continuous.cfcₙ {X : Type u_1} {𝕜 : Type u_2} {A : Type u_3} {p : AProp} [RCLike 𝕜] [NonUnitalNormedRing A] [StarRing A] [NormedSpace 𝕜 A] [IsScalarTower 𝕜 A A] [SMulCommClass 𝕜 A A] [ContinuousStar A] [NonUnitalIsometricContinuousFunctionalCalculus 𝕜 A p] [TopologicalSpace X] {s : Set 𝕜} (hs : IsCompact s) (f : 𝕜𝕜) {a : XA} (ha_cont : Continuous a) (ha : ∀ (x : X), quasispectrum 𝕜 (a x) s) (hf : ContinuousOn f s := by cfc_cont_tac) (hf0 : f 0 = 0 := by cfc_zero_tac) (ha' : ∀ (x : X), p (a x) := by cfc_tac) :
Continuous fun (x : X) => cfcₙ f (a x)

cfcₙ is continuous in the variable a : A when s : Set 𝕜 is compact and a varies over elements whose quasispectrum is contained in s, all of which satisfy the predicate p, and the function f is continuous s and f 0 = 0.

theorem continuous_cfcₙ {X : Type u_1} {𝕜 : Type u_2} {A : Type u_3} {p : AProp} [RCLike 𝕜] [NonUnitalNormedRing A] [StarRing A] [NormedSpace 𝕜 A] [IsScalarTower 𝕜 A A] [SMulCommClass 𝕜 A A] [ContinuousStar A] [NonUnitalIsometricContinuousFunctionalCalculus 𝕜 A p] [TopologicalSpace X] {s : Set 𝕜} (hs : IsCompact s) (hs0 : 0 s) (f : 𝕜𝕜) (a : XA) (ha_cont : Continuous a) (ha : ∀ (x : X), quasispectrum 𝕜 (a x) s) (hf : ContinuousOn f s := by cfc_cont_tac) (hf0 : f 0 = 0 := by cfc_zero_tac) (ha' : ∀ (x : X), p (a x) := by cfc_tac) :
Continuous fun (x : X) => cfcₙ f (a x)

cfcₙ is continuous in the variable a : A when s : Set 𝕜 is compact and a varies over elements whose spectrum is contained in s, all of which satisfy the predicate p, and the function f is continuous on the spectrum of a and maps zero to itself.

A version of continuousOn_cfcₙ over ℝ≥0 instead of RCLike 𝕜.

theorem Filter.Tendsto.cfcₙ_nnreal {X : Type u_1} {A : Type u_2} [NonUnitalNormedRing A] [StarRing A] [NormedSpace A] [IsScalarTower A A] [SMulCommClass A A] [ContinuousStar A] [NonUnitalIsometricContinuousFunctionalCalculus A IsSelfAdjoint] [PartialOrder A] [StarOrderedRing A] [NonnegSpectrumClass A] [T2Space A] [IsTopologicalRing A] {s : Set NNReal} (hs : IsCompact s) (f : NNRealNNReal) {a : XA} {a₀ : A} {l : Filter X} (ha_tendsto : Tendsto a l (nhds a₀)) (ha : ∀ᶠ (x : X) in l, quasispectrum NNReal (a x) s) (ha' : ∀ᶠ (x : X) in l, 0 a x) (ha₀ : quasispectrum NNReal a₀ s) (ha₀' : 0 a₀) (hf : ContinuousOn f s := by cfc_cont_tac) (hf0 : f 0 = 0 := by cfc_zero_tac) :
Tendsto (fun (x : X) => cfcₙ f (a x)) l (nhds (cfcₙ f a₀))

If f : ℝ≥0 → ℝ≥0 is continuous on a compact set s and f 0 = 0 and a : X → A tends to a₀ : A along a filter l (such that eventually a x satisfies the predicate p associated to ℝ≥0 and has quasispectrum contained in s, as does a₀), then fun x ↦ cfcₙ f (a x) tends to cfcₙ f a₀.

theorem ContinuousAt.cfcₙ_nnreal {X : Type u_1} {A : Type u_2} [NonUnitalNormedRing A] [StarRing A] [NormedSpace A] [IsScalarTower A A] [SMulCommClass A A] [ContinuousStar A] [NonUnitalIsometricContinuousFunctionalCalculus A IsSelfAdjoint] [PartialOrder A] [StarOrderedRing A] [NonnegSpectrumClass A] [T2Space A] [IsTopologicalRing A] [TopologicalSpace X] {s : Set NNReal} (hs : IsCompact s) (f : NNRealNNReal) {a : XA} {x₀ : X} (ha_cont : ContinuousAt a x₀) (ha : ∀ᶠ (x : X) in nhds x₀, quasispectrum NNReal (a x) s) (ha' : ∀ᶠ (x : X) in nhds x₀, 0 a x) (hf : ContinuousOn f s := by cfc_cont_tac) (hf0 : f 0 = 0 := by cfc_zero_tac) :
ContinuousAt (fun (x : X) => cfcₙ f (a x)) x₀

If f : ℝ≥0 → ℝ≥0 is continuous on a compact set s and f 0 = 0 and a : X → A is continuous at x₀, and eventually a x satisfies the predicate p associated to ℝ≥0 and has quasispectrum contained in s), then fun x ↦ cfcₙ f (a x) is continuous at x₀.

theorem ContinuousWithinAt.cfcₙ_nnreal {X : Type u_1} {A : Type u_2} [NonUnitalNormedRing A] [StarRing A] [NormedSpace A] [IsScalarTower A A] [SMulCommClass A A] [ContinuousStar A] [NonUnitalIsometricContinuousFunctionalCalculus A IsSelfAdjoint] [PartialOrder A] [StarOrderedRing A] [NonnegSpectrumClass A] [T2Space A] [IsTopologicalRing A] [TopologicalSpace X] {s : Set NNReal} (hs : IsCompact s) (f : NNRealNNReal) {a : XA} {x₀ : X} {t : Set X} (hx₀ : x₀ t) (ha_cont : ContinuousWithinAt a t x₀) (ha : ∀ᶠ (x : X) in nhdsWithin x₀ t, quasispectrum NNReal (a x) s) (ha' : ∀ᶠ (x : X) in nhdsWithin x₀ t, 0 a x) (hf : ContinuousOn f s := by cfc_cont_tac) (hf0 : f 0 = 0 := by cfc_zero_tac) :
ContinuousWithinAt (fun (x : X) => cfcₙ f (a x)) t x₀

If f : ℝ≥0 → ℝ≥0 is continuous on a compact set s and f 0 = 0 and a : X → A is continuous at x₀ within a set t : Set X, and eventually a x satisfies the predicate p associated to ℝ≥0 and has quasispectrum contained in s), then fun x ↦ cfcₙ f (a x) is continuous at x₀ within t.

theorem ContinuousOn.cfcₙ_nnreal {X : Type u_1} {A : Type u_2} [NonUnitalNormedRing A] [StarRing A] [NormedSpace A] [IsScalarTower A A] [SMulCommClass A A] [ContinuousStar A] [NonUnitalIsometricContinuousFunctionalCalculus A IsSelfAdjoint] [PartialOrder A] [StarOrderedRing A] [NonnegSpectrumClass A] [T2Space A] [IsTopologicalRing A] [TopologicalSpace X] {s : Set NNReal} (hs : IsCompact s) (f : NNRealNNReal) {a : XA} {t : Set X} (ha_cont : ContinuousOn a t) (ha : xt, quasispectrum NNReal (a x) s) (ha' : xt, 0 a x) (hf : ContinuousOn f s := by cfc_cont_tac) (hf0 : f 0 = 0 := by cfc_zero_tac) :
ContinuousOn (fun (x : X) => cfcₙ f (a x)) t

If f : ℝ≥0 → ℝ≥0 is continuous on a compact set s and f 0 = 0 and a : X → A is continuous on t : Set X, and a x satisfies the predicate p associated to ℝ≥0 and has quasispectrum contained in s for all x ∈ t, then fun x ↦ cfcₙ f (a x) is continuous on t.

theorem Continuous.cfcₙ_nnreal {X : Type u_1} {A : Type u_2} [NonUnitalNormedRing A] [StarRing A] [NormedSpace A] [IsScalarTower A A] [SMulCommClass A A] [ContinuousStar A] [NonUnitalIsometricContinuousFunctionalCalculus A IsSelfAdjoint] [PartialOrder A] [StarOrderedRing A] [NonnegSpectrumClass A] [T2Space A] [IsTopologicalRing A] [TopologicalSpace X] {s : Set NNReal} (hs : IsCompact s) (f : NNRealNNReal) {a : XA} (ha_cont : Continuous a) (ha : ∀ (x : X), quasispectrum NNReal (a x) s) (hf : ContinuousOn f s := by cfc_cont_tac) (hf0 : f 0 = 0 := by cfc_zero_tac) (ha' : ∀ (x : X), 0 a x := by cfc_tac) :
Continuous fun (x : X) => cfcₙ f (a x)

cfcₙ is continuous in the variable a : A when s : Set ℝ≥0 is compact and a varies over elements whose quasispectrum is contained in s, all of which satisfy the predicate p, and the function f is continuous s and f 0 = 0.