Topology of pointwise convergence on continous linear maps #
Main definitions #
PointwiseConvergenceCLM: Type synonym ofE →SL[σ] Fequipped with the uniform convergence topology on finite sets.PointwiseConvergenceCLM.evalCLM: The evaluation map(f : E →SLₚₜ[σ] F) ↦ f afor fixeda : Eas a continuous linear map.ContinousLinearMap.toPointwiseConvergenceCLM: The canonical map fromE →SL[σ] FtoE →SLₚₜ[σ] Fas a continuous linear map. This is the statement that bounded convergence is stronger than pointwise convergence.PointwiseConvergenceCLM.equivWeakDual: The continuous equivalence betweenE →Lₚₜ[𝕜] 𝕜andWeakDual 𝕜 E.
Main statements #
PointwiseConvergenceCLM.tendsto_iff_forall_tendsto: In the topology of pointwise convergence,aconverges toa₀iff for everyx : Ethe mapa · xconverges toa₀ x.PointwiseConvergenceCLM.continuous_of_continuous_eval: A map tog : α → E →SLₚₜ[σ] Fis continuous if for everyx : Ethe evaluationg · xis continuous.
Notation #
E →SLₚₜ[σ] Fis space of continuous linear maps equipped with pointwise convergence topology.
Topology of pointwise convergence #
The space of continuous linear maps equipped with the topology of pointwise convergence, sometimes also called the strong operator topology. We avoid this terminology since so many other things share similar names, and using "pointwise convergence" in the name is more informative.
This topology is also known as the weak*-topology in the case that σ = RingHom.id 𝕜 and F = 𝕜
Instances For
The space of continuous linear maps equipped with the topology of pointwise convergence, sometimes also called the strong operator topology. We avoid this terminology since so many other things share similar names, and using "pointwise convergence" in the name is more informative.
This topology is also known as the weak*-topology in the case that σ = RingHom.id 𝕜 and F = 𝕜
Equations
- One or more equations did not get rendered due to their size.
Instances For
The space of continuous linear maps equipped with the topology of pointwise convergence, sometimes also called the strong operator topology. We avoid this terminology since so many other things share similar names, and using "pointwise convergence" in the name is more informative.
This topology is also known as the weak*-topology in the case that σ = RingHom.id 𝕜 and F = 𝕜
Equations
- One or more equations did not get rendered due to their size.
Instances For
In the topology of pointwise convergence, a converges to a₀ iff for every x : E the map
a · x converges to a₀ x.
Coercion from E →SLₚₜ[σ] F to E →ₛₗ[σ] F as a 𝕜₂-linear map.
Equations
Instances For
Coercion from E →Lₚₜ[𝕜] F to E →ₗ[𝕜] F as a 𝕜-linear map.
Equations
Instances For
The evaluation map (f : E →SLₚₜ[σ] F) ↦ f a for a : E as a continuous linear map.
Equations
- PointwiseConvergenceCLM.evalCLM σ F a = { toLinearMap := (PointwiseConvergenceCLM.coeLMₛₗ σ E F).flip a, cont := ⋯ }
Instances For
A map to E →SLₚₜ[σ] F is continuous if for every x : E the evaluation g · x is
continuous.
The topology of bounded convergence is stronger than the topology of pointwise convergence.
Equations
- ContinuousLinearMap.toPointwiseConvergenceCLM 𝕜₂ σ E F = { toLinearMap := LinearMap.id, cont := ⋯ }
Instances For
The topology of pointwise convergence on E →Lₚₜ[𝕜] 𝕜 coincides with the weak-* topology.
Equations
- PointwiseConvergenceCLM.equivWeakDual 𝕜 E = { toLinearEquiv := LinearEquiv.refl 𝕜 (E →L[𝕜] 𝕜), continuous_toFun := ⋯, continuous_invFun := ⋯ }