Multiplier Algebra of a C⋆-algebra #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
Define the multiplier algebra of a C⋆-algebra as the algebra (over 𝕜
) of double centralizers,
for which we provide the localized notation 𝓜(𝕜, A)
. A double centralizer is a pair of
continuous linear maps L R : A →L[𝕜] A
satisfying the intertwining condition R x * y = x * L y
.
There is a natural embedding A → 𝓜(𝕜, A)
which sends a : A
to the continuous linear maps
L R : A →L[𝕜] A
given by left and right multiplication by a
, and we provide this map as a
coercion.
The multiplier algebra corresponds to a non-commutative Stone–Čech compactification in the sense
that when the algebra A
is commutative, it can be identified with C₀(X, ℂ)
for some locally
compact Hausdorff space X
, and in that case 𝓜(𝕜, A)
can be identified with C(β X, ℂ)
.
Implementation notes #
We make the hypotheses on 𝕜
as weak as possible so that, in particular, this construction works
for both 𝕜 = ℝ
and 𝕜 = ℂ
.
The reader familiar with C⋆-algebra theory may recognize that one
only needs L
and R
to be functions instead of continuous linear maps, at least when A
is a
C⋆-algebra. Our intention is simply to eventually provide a constructor for this situation.
We pull back the normed_algebra
structure (and everything contained therein) through the
ring (even algebra) homomorphism
double_centralizer.to_prod_mul_opposite_hom : 𝓜(𝕜, A) →+* (A →L[𝕜] A) × (A →L[𝕜] A)ᵐᵒᵖ
which
sends a : 𝓜(𝕜, A)
to (a.fst, mul_opposite.op a.snd)
. The star structure is provided
separately.
References #
TODO #
- Define a type synonym for
𝓜(𝕜, A)
which is equipped with the strict uniform space structure and show it is complete - Show that the image of
A
in𝓜(𝕜, A)
is an essential ideal - Prove the universal property of
𝓜(𝕜, A)
- Construct a double centralizer from a pair of maps (not necessarily linear or continuous)
L : A → A
,R : A → A
satisfying the centrality condition∀ x y, R x * y = x * L y
. - Show that if
A
is unital, thenA ≃⋆ₐ[𝕜] 𝓜(𝕜, A)
.
- to_prod : (A →L[𝕜] A) × (A →L[𝕜] A)
- central : ∀ (x y : A), ⇑(self.to_prod.snd) x * y = x * ⇑(self.to_prod.fst) y
The type of double centralizers, also known as the multiplier algebra and denoted by
𝓜(𝕜, A)
, of a non-unital normed algebra.
If x : 𝓜(𝕜, A)
, then x.fst
and x.snd
are what is usually referred to as $L$ and $R$.
Instances for double_centralizer
- double_centralizer.has_sizeof_inst
- double_centralizer.has_add
- double_centralizer.has_zero
- double_centralizer.has_neg
- double_centralizer.has_sub
- double_centralizer.has_smul
- double_centralizer.is_scalar_tower
- double_centralizer.smul_comm_class
- double_centralizer.is_central_scalar
- double_centralizer.has_one
- double_centralizer.has_mul
- double_centralizer.has_nat_cast
- double_centralizer.has_int_cast
- double_centralizer.nat.has_pow
- double_centralizer.inhabited
- double_centralizer.ring
- double_centralizer.module
- double_centralizer.algebra
- double_centralizer.has_star
- double_centralizer.star_add_monoid
- double_centralizer.star_ring
- double_centralizer.star_module
- double_centralizer.has_coe_t
- double_centralizer.normed_ring
- double_centralizer.normed_space
- double_centralizer.normed_algebra
- double_centralizer.complete_space
- double_centralizer.cstar_ring
Algebraic structure #
Because the multiplier algebra is defined as the algebra of double centralizers, there is a natural
injection double_centralizer.to_prod_mul_opposite : 𝓜(𝕜, A) → (A →L[𝕜] A) × (A →L[𝕜] A)ᵐᵒᵖ
defined by λ a, (a.fst, mul_opposite.op a.snd)
. We use this map to pull back the ring, module and
algebra structure from (A →L[𝕜] A) × (A →L[𝕜] A)ᵐᵒᵖ
to 𝓜(𝕜, A)
.
Equations
- double_centralizer.has_neg = {neg := λ (a : double_centralizer 𝕜 A), {to_prod := -a.to_prod, central := _}}
Equations
- double_centralizer.has_smul = {smul := λ (s : S) (a : double_centralizer 𝕜 A), {to_prod := s • a.to_prod, central := _}}
Equations
The natural injection from double_centralizer.to_prod
except the second coordinate inherits
mul_opposite.op
. The ring structure on 𝓜(𝕜, A)
is the pullback under this map.
Equations
- double_centralizer.to_prod_mul_opposite = λ (a : double_centralizer 𝕜 A), (a.to_prod.fst, mul_opposite.op a.to_prod.snd)
The ring structure is inherited as the pullback under the injective map
double_centralizer.to_prod_mul_opposite : 𝓜(𝕜, A) → (A →L[𝕜] A) × (A →L[𝕜] A)ᵐᵒᵖ
Equations
- double_centralizer.ring = function.injective.ring double_centralizer.to_prod_mul_opposite double_centralizer.to_prod_mul_opposite_injective double_centralizer.ring._proof_10 double_centralizer.ring._proof_11 double_centralizer.ring._proof_12 double_centralizer.ring._proof_13 double_centralizer.ring._proof_14 double_centralizer.ring._proof_15 double_centralizer.ring._proof_16 double_centralizer.ring._proof_17 double_centralizer.ring._proof_18 double_centralizer.ring._proof_19 double_centralizer.ring._proof_20
The canonical map double_centralizer.to_prod
as an additive group homomorphism.
Equations
- double_centralizer.to_prod_hom = {to_fun := double_centralizer.to_prod _inst_5, map_zero' := _, map_add' := _}
The canonical map double_centralizer.to_prod_mul_opposite
as a ring homomorphism.
Equations
- double_centralizer.to_prod_mul_opposite_hom = {to_fun := double_centralizer.to_prod_mul_opposite _inst_5, map_one' := _, map_mul' := _, map_zero' := _, map_add' := _}
The module structure is inherited as the pullback under the additive group monomorphism
double_centralizer.to_prod : 𝓜(𝕜, A) →+ (A →L[𝕜] A) × (A →L[𝕜] A)
Equations
- double_centralizer.module = function.injective.module S double_centralizer.to_prod_hom double_centralizer.ext double_centralizer.module._proof_3
Equations
- double_centralizer.algebra = {to_has_smul := double_centralizer.has_smul _inst_4, to_ring_hom := {to_fun := λ (k : 𝕜), {to_prod := ⇑(algebra_map 𝕜 ((A →L[𝕜] A) × (A →L[𝕜] A))) k, central := _}, map_one' := _, map_mul' := _, map_zero' := _, map_add' := _}, commutes' := _, smul_def' := _}
Star structure #
The star operation on a : 𝓜(𝕜, A)
is given by
(star a).to_prod = (star ∘ a.snd ∘ star, star ∘ a.fst ∘ star)
.
Equations
Coercion from an algebra into its multiplier algebra #
The natural coercion of A
into 𝓜(𝕜, A)
given by sending a : A
to the pair of linear
maps Lₐ Rₐ : A →L[𝕜] A
given by left- and right-multiplication by a
, respectively.
Warning: if A = 𝕜
, then this is a coercion which is not definitionally equal to the
algebra_map 𝕜 𝓜(𝕜, 𝕜)
coercion, but these are propositionally equal. See
double_centralizer.coe_eq_algebra_map
below.
Equations
- double_centralizer.has_coe_t = {coe := λ (a : A), {to_prod := (⇑(continuous_linear_map.mul 𝕜 A) a, ⇑((continuous_linear_map.mul 𝕜 A).flip) a), central := _}}
The coercion of an algebra into its multiplier algebra as a non-unital star algebra homomorphism.
Norm structures #
We define the norm structure on 𝓜(𝕜, A)
as the pullback under
double_centralizer.to_prod_mul_opposite_hom : 𝓜(𝕜, A) →+* (A →L[𝕜] A) × (A →L[𝕜] A)ᵐᵒᵖ
, which
provides a definitional isometric embedding. Consequently, completeness of 𝓜(𝕜, A)
is obtained
by proving that the range of this map is closed.
In addition, we prove that 𝓜(𝕜, A)
is a normed algebra, and, when A
is a C⋆-algebra, we show
that 𝓜(𝕜, A)
is also a C⋆-algebra. Moreover, in this case, for a : 𝓜(𝕜, A)
,
‖a‖ = ‖a.fst‖ = ‖a.snd‖
.
The normed group structure is inherited as the pullback under the ring monomoprhism
double_centralizer.to_prod_mul_opposite_hom : 𝓜(𝕜, A) →+* (A →L[𝕜] A) × (A →L[𝕜] A)ᵐᵒᵖ
.
Equations
Equations
For a : 𝓜(𝕜, A)
, the norms of a.fst
and a.snd
coincide, and hence these
also coincide with ‖a‖
which is max (‖a.fst‖) (‖a.snd‖)
.