mathlib documentation

algebra.star.self_adjoint

Self-adjoint elements of a star additive group #

This file defines self_adjoint R, where R is a star additive monoid, as the additive subgroup containing the elements that satisfy star x = x. This includes, for instance, Hermitian operators on Hilbert spaces.

Implementation notes #

TODO #

def self_adjoint (R : Type u_1) [add_group R] [star_add_monoid R] :

The self-adjoint elements of a star additive group, as an additive subgroup.

Equations
theorem self_adjoint.mem_iff {R : Type u_1} [add_group R] [star_add_monoid R] {x : R} :
@[simp, norm_cast]
theorem self_adjoint.star_coe_eq {R : Type u_1} [add_group R] [star_add_monoid R] {x : (self_adjoint R)} :
@[protected, instance]
Equations
@[protected, instance]
def self_adjoint.has_one {R : Type u_1} [ring R] [star_ring R] :
Equations
@[simp, norm_cast]
theorem self_adjoint.coe_one {R : Type u_1} [ring R] [star_ring R] :
1 = 1
@[protected, instance]
theorem self_adjoint.one_mem {R : Type u_1} [ring R] [star_ring R] :
theorem self_adjoint.bit0_mem {R : Type u_1} [ring R] [star_ring R] {x : R} (hx : x self_adjoint R) :
theorem self_adjoint.bit1_mem {R : Type u_1} [ring R] [star_ring R] {x : R} (hx : x self_adjoint R) :
theorem self_adjoint.conjugate {R : Type u_1} [ring R] [star_ring R] {x : R} (hx : x self_adjoint R) (z : R) :
(z * x) * star z self_adjoint R
theorem self_adjoint.conjugate' {R : Type u_1} [ring R] [star_ring R] {x : R} (hx : x self_adjoint R) (z : R) :
((star z) * x) * z self_adjoint R
@[protected, instance]
def self_adjoint.has_mul {R : Type u_1} [comm_ring R] [star_ring R] :
Equations
@[simp, norm_cast]
theorem self_adjoint.coe_mul {R : Type u_1} [comm_ring R] [star_ring R] (x y : (self_adjoint R)) :
x * y = (x) * y
@[protected, instance]
def self_adjoint.field {R : Type u_1} [field R] [star_ring R] :
Equations
@[simp, norm_cast]
theorem self_adjoint.coe_inv {R : Type u_1} [field R] [star_ring R] (x : (self_adjoint R)) :
@[protected, instance]
def self_adjoint.has_scalar {R : Type u_1} {A : Type u_2} [semiring R] [has_star R] [has_trivial_star R] [add_comm_group A] [star_add_monoid A] [module R A] [star_module R A] :
Equations
@[simp, norm_cast]
theorem self_adjoint.coe_smul {R : Type u_1} {A : Type u_2} [semiring R] [has_star R] [has_trivial_star R] [add_comm_group A] [star_add_monoid A] [module R A] [star_module R A] (r : R) (x : (self_adjoint A)) :
(r x) = r x
@[protected, instance]
def self_adjoint.mul_action {R : Type u_1} {A : Type u_2} [semiring R] [has_star R] [has_trivial_star R] [add_comm_group A] [star_add_monoid A] [module R A] [star_module R A] :
Equations
@[protected, instance]
def self_adjoint.module {R : Type u_1} {A : Type u_2} [semiring R] [has_star R] [has_trivial_star R] [add_comm_group A] [star_add_monoid A] [module R A] [star_module R A] :
Equations