mathlib3 documentation

analysis.normed_space.star.basic

Normed star rings and algebras #

THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.

A normed star group is a normed group with a compatible star which is isometric.

A C⋆-ring is a normed star group that is also a ring and that verifies the stronger condition ‖x⋆ * x‖ = ‖x‖^2 for all x. If a C⋆-ring is also a star algebra, then it is a C⋆-algebra.

To get a C⋆-algebra E over field 𝕜, use [normed_field 𝕜] [star_ring 𝕜] [normed_ring E] [star_ring E] [cstar_ring E] [normed_algebra 𝕜 E] [star_module 𝕜 E].

TODO #

The star map in a normed star group is a normed group homomorphism.

Equations

The star map in a normed star group is an isometry

@[protected, instance]
@[protected, instance]

In a C*-ring, star preserves the norm.

@[simp]
@[simp]
@[protected, instance]
def pi.star_ring' {ι : Type u_4} {R : ι Type u_7} [Π (i : ι), non_unital_normed_ring (R i)] [Π (i : ι), star_ring (R i)] :
star_ring (Π (i : ι), R i)

This instance exists to short circuit type class resolution because of problems with inference involving Π-types.

Equations
@[protected, instance]
def prod.cstar_ring {R₁ : Type u_5} {R₂ : Type u_6} [non_unital_normed_ring R₁] [star_ring R₁] [cstar_ring R₁] [non_unital_normed_ring R₂] [star_ring R₂] [cstar_ring R₂] :
cstar_ring (R₁ × R₂)
@[protected, instance]
def pi.cstar_ring {ι : Type u_4} {R : ι Type u_7} [Π (i : ι), non_unital_normed_ring (R i)] [Π (i : ι), star_ring (R i)] [fintype ι] [ (i : ι), cstar_ring (R i)] :
cstar_ring (Π (i : ι), R i)
@[protected, instance]
def pi.cstar_ring' {ι : Type u_4} {R₁ : Type u_5} [non_unital_normed_ring R₁] [star_ring R₁] [cstar_ring R₁] [fintype ι] :
cstar_ring R₁)
@[simp]
theorem cstar_ring.norm_one {E : Type u_2} [normed_ring E] [star_ring E] [cstar_ring E] [nontrivial E] :
@[protected, instance]
@[simp]
theorem cstar_ring.norm_of_mem_unitary {E : Type u_2} [normed_ring E] [star_ring E] [cstar_ring E] [nontrivial E] {U : E} (hU : U unitary E) :
@[simp]
theorem cstar_ring.norm_coe_unitary_mul {E : Type u_2} [normed_ring E] [star_ring E] [cstar_ring E] (U : (unitary E)) (A : E) :
@[simp]
theorem cstar_ring.norm_unitary_smul {E : Type u_2} [normed_ring E] [star_ring E] [cstar_ring E] (U : (unitary E)) (A : E) :
theorem cstar_ring.norm_mem_unitary_mul {E : Type u_2} [normed_ring E] [star_ring E] [cstar_ring E] {U : E} (A : E) (hU : U unitary E) :
@[simp]
theorem cstar_ring.norm_mul_coe_unitary {E : Type u_2} [normed_ring E] [star_ring E] [cstar_ring E] (A : E) (U : (unitary E)) :
theorem cstar_ring.norm_mul_mem_unitary {E : Type u_2} [normed_ring E] [star_ring E] [cstar_ring E] (A : E) {U : E} (hU : U unitary E) :
theorem is_self_adjoint.nnnorm_pow_two_pow {E : Type u_2} [normed_ring E] [star_ring E] [cstar_ring E] {x : E} (hx : is_self_adjoint x) (n : ) :
x ^ 2 ^ n‖₊ = x‖₊ ^ 2 ^ n
theorem self_adjoint.nnnorm_pow_two_pow {E : Type u_2} [normed_ring E] [star_ring E] [cstar_ring E] (x : (self_adjoint E)) (n : ) :
x ^ 2 ^ n‖₊ = x‖₊ ^ 2 ^ n
def starₗᵢ (𝕜 : Type u_1) {E : Type u_2} [comm_semiring 𝕜] [star_ring 𝕜] [seminormed_add_comm_group E] [star_add_monoid E] [normed_star_group E] [module 𝕜 E] [star_module 𝕜 E] :

star bundled as a linear isometric equivalence

Equations
@[simp]
theorem coe_starₗᵢ {𝕜 : Type u_1} {E : Type u_2} [comm_semiring 𝕜] [star_ring 𝕜] [seminormed_add_comm_group E] [star_add_monoid E] [normed_star_group E] [module 𝕜 E] [star_module 𝕜 E] :
theorem starₗᵢ_apply {𝕜 : Type u_1} {E : Type u_2} [comm_semiring 𝕜] [star_ring 𝕜] [seminormed_add_comm_group E] [star_add_monoid E] [normed_star_group E] [module 𝕜 E] [star_module 𝕜 E] {x : E} :
@[protected, instance]
def star_subalgebra.to_normed_algebra {𝕜 : Type u_1} {A : Type u_2} [normed_field 𝕜] [star_ring 𝕜] [semi_normed_ring A] [star_ring A] [normed_algebra 𝕜 A] [star_module 𝕜 A] (S : star_subalgebra 𝕜 A) :
Equations
@[protected, instance]