The partial order on matrices #
This file constructs the partial order and star ordered instances on matrices on π
.
This allows us to use more general results from Cβ-algebras, like CFC.sqrt
.
Main results #
Matrix.instPartialOrder
: the partial order on matrices given byx β€ y := (y - x).PosSemidef
.Matrix.PosSemidef.dotProduct_mulVec_zero_iff
: for a positive semi-definite matrixA
, we havexβ A x = 0
iffA x = 0
.Matrix.PosDef.matrixInnerProductSpace
: the inner product on matrices induced by a positive definite matrixM
:βͺx, yβ« = (y * M * xα΄΄).trace
.
Implementation notes #
Note that the partial order instance is scoped to MatrixOrder
.
Please open scoped MatrixOrder
to use this.
The preorder on matrices given by A β€ B := (B - A).PosSemidef
.
Equations
- Matrix.instPreOrder = { le := fun (A B : Matrix n n π) => (B - A).PosSemidef, le_refl := β―, le_trans := β―, lt_iff_le_not_ge := β― }
Instances For
Alias of the forward direction of Matrix.nonneg_iff_posSemidef
.
Alias of the reverse direction of Matrix.nonneg_iff_posSemidef
.
The partial order on matrices given by A β€ B := (B - A).PosSemidef
.
Equations
- Matrix.instPartialOrder = { toPreorder := Matrix.instPreOrder, le_antisymm := β― }
Instances For
The positive semidefinite square root of a positive semidefinite matrix
Equations
- hA.sqrt = ββ―.eigenvectorUnitary * Matrix.diagonal (RCLike.ofReal β (fun (x : β) => βx) β β―.eigenvalues) * star ββ―.eigenvectorUnitary
Instances For
Alias of the forward direction of CFC.sq_eq_sq_iff
.
For A
positive semidefinite, we have xβ A x = 0
iff A x = 0
(linear maps version).
A matrix is positive semidefinite if and only if it has the form Bα΄΄ * B
for some B
.
Alias of CStarAlgebra.nonneg_iff_eq_star_mul_self
.
A positive semi-definite matrix is positive definite if and only if it is invertible.
A matrix is positive definite if and only if it has the form Bα΄΄ * B
for some invertible B
.
Alias of Matrix.posDef_iff_eq_conjTranspose_mul_self
.
A matrix is positive definite if and only if it has the form Bα΄΄ * B
for some invertible B
.
A positive definite matrix M
induces a norm on Matrix n n π
:
βxβ = sqrt (x * M * xα΄΄).trace
.
Instances For
A positive definite matrix M
induces an inner product on Matrix n n π
:
βͺx, yβ« = (y * M * xα΄΄).trace
.
Equations
- One or more equations did not get rendered due to their size.