Hermitian matrices #
This file defines Hermitian matrices and some basic results about them.
See also IsSelfAdjoint, which generalizes this definition to other star rings.
Main definition #
Matrix.IsHermitian: a matrixA : Matrix n n αis Hermitian ifAᴴ = A.
Tags #
self-adjoint matrix, hermitian matrix
A matrix is Hermitian if it is equal to its conjugate transpose. On the reals, this definition captures symmetric matrices.
Equations
- A.IsHermitian = (A.conjTranspose = A)
Instances For
Equations
Alias of the reverse direction of Matrix.isHermitian_iff_isSelfAdjoint.
Alias of the forward direction of Matrix.isHermitian_iff_isSelfAdjoint.
A block matrix A.from_blocks B C D is Hermitian,
if A and D are Hermitian and Bᴴ = C.
This is the iff version of Matrix.IsHermitian.fromBlocks.
A diagonal matrix is Hermitian if the entries are self-adjoint (as a vector)
A diagonal matrix is Hermitian if each diagonal entry is self-adjoint
A diagonal matrix is Hermitian if the entries have the trivial star operation
(such as on the reals).
Note this is more general than IsSelfAdjoint.mul_star_self as B can be rectangular.
Note this is more general than IsSelfAdjoint.star_mul_self as B can be rectangular.
Note this is more general than IsSelfAdjoint.conjugate' as B can be rectangular.
Note this is more general than IsSelfAdjoint.conjugate as B can be rectangular.
Alias of Matrix.IsHermitian.commute_iff.
Note this is more general for matrices than isSelfAdjoint_one as it does not
require Fintype n, which is necessary for Monoid (Matrix n n R).
Note that IsSelfAdjoint.zpow does not apply to matrices as they are not a division ring.
Notation for Sum.elim, scoped within the Matrix namespace.
Equations
- Matrix.«term_⊕ᵥ_» = Lean.ParserDescr.trailingNode `Matrix.«term_⊕ᵥ_» 65 65 (Lean.ParserDescr.binary `andthen (Lean.ParserDescr.symbol " ⊕ᵥ ") (Lean.ParserDescr.cat `term 66))
Instances For
The diagonal elements of a complex Hermitian matrix are real.
A matrix is Hermitian iff the corresponding linear map is self adjoint.