Documentation

Mathlib.LinearAlgebra.Matrix.PosDef

Positive Definite Matrices #

This file defines positive (semi)definite matrices and connects the notion to positive definiteness of quadratic forms. Most results require π•œ = ℝ or β„‚.

Main definitions #

##Β Main results

Positive semidefinite matrices #

def Matrix.PosSemidef {n : Type u_2} {R : Type u_3} [Fintype n] [CommRing R] [PartialOrder R] [StarRing R] [StarOrderedRing R] (M : Matrix n n R) :

A matrix M : Matrix n n R is positive semidefinite if it is Hermitian and xα΄΄ * M * x is nonnegative for all x.

Equations
Instances For
    theorem Matrix.posSemidef_diagonal_iff {n : Type u_2} {R : Type u_3} [Fintype n] [CommRing R] [PartialOrder R] [StarRing R] [StarOrderedRing R] [DecidableEq n] {d : n β†’ R} :
    (Matrix.diagonal d).PosSemidef ↔ βˆ€ (i : n), 0 ≀ d i

    A diagonal matrix is positive semidefinite iff its diagonal entries are nonnegative.

    theorem Matrix.PosSemidef.isHermitian {n : Type u_2} {R : Type u_3} [Fintype n] [CommRing R] [PartialOrder R] [StarRing R] [StarOrderedRing R] {M : Matrix n n R} (hM : M.PosSemidef) :
    M.IsHermitian
    theorem Matrix.PosSemidef.re_dotProduct_nonneg {n : Type u_2} {π•œ : Type u_4} [Fintype n] [RCLike π•œ] {M : Matrix n n π•œ} (hM : M.PosSemidef) (x : n β†’ π•œ) :
    0 ≀ RCLike.re (Matrix.dotProduct (star x) (M.mulVec x))
    theorem Matrix.PosSemidef.conjTranspose_mul_mul_same {n : Type u_2} {R : Type u_3} [Fintype n] [CommRing R] [PartialOrder R] [StarRing R] [StarOrderedRing R] {A : Matrix n n R} (hA : A.PosSemidef) {m : Type u_5} [Fintype m] (B : Matrix n m R) :
    (B.conjTranspose * A * B).PosSemidef
    theorem Matrix.PosSemidef.mul_mul_conjTranspose_same {n : Type u_2} {R : Type u_3} [Fintype n] [CommRing R] [PartialOrder R] [StarRing R] [StarOrderedRing R] {A : Matrix n n R} (hA : A.PosSemidef) {m : Type u_5} [Fintype m] (B : Matrix m n R) :
    (B * A * B.conjTranspose).PosSemidef
    theorem Matrix.PosSemidef.submatrix {m : Type u_1} {n : Type u_2} {R : Type u_3} [Fintype m] [Fintype n] [CommRing R] [PartialOrder R] [StarRing R] [StarOrderedRing R] {M : Matrix n n R} (hM : M.PosSemidef) (e : m β†’ n) :
    (M.submatrix e e).PosSemidef
    theorem Matrix.PosSemidef.transpose {n : Type u_2} {R : Type u_3} [Fintype n] [CommRing R] [PartialOrder R] [StarRing R] [StarOrderedRing R] {M : Matrix n n R} (hM : M.PosSemidef) :
    M.transpose.PosSemidef
    theorem Matrix.PosSemidef.conjTranspose {n : Type u_2} {R : Type u_3} [Fintype n] [CommRing R] [PartialOrder R] [StarRing R] [StarOrderedRing R] {M : Matrix n n R} (hM : M.PosSemidef) :
    M.conjTranspose.PosSemidef
    theorem Matrix.PosSemidef.pow {n : Type u_2} {R : Type u_3} [Fintype n] [CommRing R] [PartialOrder R] [StarRing R] [StarOrderedRing R] [DecidableEq n] {M : Matrix n n R} (hM : M.PosSemidef) (k : β„•) :
    (M ^ k).PosSemidef
    theorem Matrix.PosSemidef.inv {n : Type u_2} {R : Type u_3} [Fintype n] [CommRing R] [PartialOrder R] [StarRing R] [StarOrderedRing R] [DecidableEq n] {M : Matrix n n R} (hM : M.PosSemidef) :
    M⁻¹.PosSemidef
    theorem Matrix.PosSemidef.zpow {n : Type u_2} {R : Type u_3} [Fintype n] [CommRing R] [PartialOrder R] [StarRing R] [StarOrderedRing R] [DecidableEq n] {M : Matrix n n R} (hM : M.PosSemidef) (z : β„€) :
    (M ^ z).PosSemidef
    theorem Matrix.PosSemidef.eigenvalues_nonneg {n : Type u_2} {π•œ : Type u_4} [Fintype n] [RCLike π•œ] [DecidableEq n] {A : Matrix n n π•œ} (hA : A.PosSemidef) (i : n) :
    0 ≀ β‹―.eigenvalues i

    The eigenvalues of a positive semi-definite matrix are non-negative

    noncomputable def Matrix.PosSemidef.sqrt {n : Type u_2} {π•œ : Type u_4} [Fintype n] [RCLike π•œ] [DecidableEq n] {A : Matrix n n π•œ} (hA : A.PosSemidef) :
    Matrix n n π•œ

    The positive semidefinite square root of a positive semidefinite matrix

    Equations
    Instances For

      Custom elaborator to produce output like (_ : PosSemidef A).sqrt in the goal view.

      Equations
      • One or more equations did not get rendered due to their size.
      Instances For
        theorem Matrix.PosSemidef.posSemidef_sqrt {n : Type u_2} {π•œ : Type u_4} [Fintype n] [RCLike π•œ] [DecidableEq n] {A : Matrix n n π•œ} (hA : A.PosSemidef) :
        hA.sqrt.PosSemidef
        @[simp]
        theorem Matrix.PosSemidef.sq_sqrt {n : Type u_2} {π•œ : Type u_4} [Fintype n] [RCLike π•œ] [DecidableEq n] {A : Matrix n n π•œ} (hA : A.PosSemidef) :
        hA.sqrt ^ 2 = A
        @[simp]
        theorem Matrix.PosSemidef.sqrt_mul_self {n : Type u_2} {π•œ : Type u_4} [Fintype n] [RCLike π•œ] [DecidableEq n] {A : Matrix n n π•œ} (hA : A.PosSemidef) :
        hA.sqrt * hA.sqrt = A
        theorem Matrix.PosSemidef.eq_of_sq_eq_sq {n : Type u_2} {π•œ : Type u_4} [Fintype n] [RCLike π•œ] [DecidableEq n] {A : Matrix n n π•œ} (hA : A.PosSemidef) {B : Matrix n n π•œ} (hB : B.PosSemidef) (hAB : A ^ 2 = B ^ 2) :
        A = B
        theorem Matrix.PosSemidef.sqrt_sq {n : Type u_2} {π•œ : Type u_4} [Fintype n] [RCLike π•œ] [DecidableEq n] {A : Matrix n n π•œ} (hA : A.PosSemidef) :
        (β‹― : (A ^ 2).PosSemidef).sqrt = A
        theorem Matrix.PosSemidef.eq_sqrt_of_sq_eq {n : Type u_2} {π•œ : Type u_4} [Fintype n] [RCLike π•œ] [DecidableEq n] {A : Matrix n n π•œ} (hA : A.PosSemidef) {B : Matrix n n π•œ} (hB : B.PosSemidef) (hAB : A ^ 2 = B) :
        A = hB.sqrt
        @[simp]
        theorem Matrix.posSemidef_submatrix_equiv {m : Type u_1} {n : Type u_2} {R : Type u_3} [Fintype m] [Fintype n] [CommRing R] [PartialOrder R] [StarRing R] [StarOrderedRing R] {M : Matrix n n R} (e : m ≃ n) :
        (M.submatrix ⇑e ⇑e).PosSemidef ↔ M.PosSemidef
        theorem Matrix.posSemidef_conjTranspose_mul_self {m : Type u_1} {n : Type u_2} {R : Type u_3} [Fintype m] [Fintype n] [CommRing R] [PartialOrder R] [StarRing R] [StarOrderedRing R] (A : Matrix m n R) :
        (A.conjTranspose * A).PosSemidef

        The conjugate transpose of a matrix mulitplied by the matrix is positive semidefinite

        theorem Matrix.posSemidef_self_mul_conjTranspose {m : Type u_1} {n : Type u_2} {R : Type u_3} [Fintype m] [Fintype n] [CommRing R] [PartialOrder R] [StarRing R] [StarOrderedRing R] (A : Matrix m n R) :
        (A * A.conjTranspose).PosSemidef

        A matrix multiplied by its conjugate transpose is positive semidefinite

        theorem Matrix.eigenvalues_conjTranspose_mul_self_nonneg {m : Type u_1} {n : Type u_2} {π•œ : Type u_4} [Fintype m] [Fintype n] [RCLike π•œ] (A : Matrix m n π•œ) [DecidableEq n] (i : n) :
        0 ≀ β‹―.eigenvalues i
        theorem Matrix.eigenvalues_self_mul_conjTranspose_nonneg {m : Type u_1} {n : Type u_2} {π•œ : Type u_4} [Fintype m] [Fintype n] [RCLike π•œ] (A : Matrix m n π•œ) [DecidableEq m] (i : m) :
        0 ≀ β‹―.eigenvalues i
        theorem Matrix.posSemidef_iff_eq_transpose_mul_self {n : Type u_2} {π•œ : Type u_4} [Fintype n] [RCLike π•œ] {A : Matrix n n π•œ} :
        A.PosSemidef ↔ βˆƒ (B : Matrix n n π•œ), A = B.conjTranspose * B

        A matrix is positive semidefinite if and only if it has the form Bα΄΄ * B for some B.

        theorem Matrix.IsHermitian.posSemidef_of_eigenvalues_nonneg {n : Type u_2} {π•œ : Type u_4} [Fintype n] [RCLike π•œ] [DecidableEq n] {A : Matrix n n π•œ} (hA : A.IsHermitian) (h : βˆ€ (i : n), 0 ≀ hA.eigenvalues i) :
        A.PosSemidef
        theorem Matrix.PosSemidef.dotProduct_mulVec_zero_iff {n : Type u_2} {π•œ : Type u_4} [Fintype n] [RCLike π•œ] {A : Matrix n n π•œ} (hA : A.PosSemidef) (x : n β†’ π•œ) :
        Matrix.dotProduct (star x) (A.mulVec x) = 0 ↔ A.mulVec x = 0

        For A positive semidefinite, we have x⋆ A x = 0 iff A x = 0.

        theorem Matrix.PosSemidef.toLinearMapβ‚‚'_zero_iff {n : Type u_2} {π•œ : Type u_4} [Fintype n] [RCLike π•œ] [DecidableEq n] {A : Matrix n n π•œ} (hA : A.PosSemidef) (x : n β†’ π•œ) :
        ((Matrix.toLinearMapβ‚‚' A) (star x)) x = 0 ↔ (Matrix.toLin' A) x = 0

        For A positive semidefinite, we have x⋆ A x = 0 iff A x = 0 (linear maps version).

        Positive definite matrices #

        def Matrix.PosDef {n : Type u_2} {R : Type u_3} [Fintype n] [CommRing R] [PartialOrder R] [StarRing R] [StarOrderedRing R] (M : Matrix n n R) :

        A matrix M : Matrix n n R is positive definite if it is hermitian and xα΄΄Mx is greater than zero for all nonzero x.

        Equations
        Instances For
          theorem Matrix.PosDef.isHermitian {n : Type u_2} {R : Type u_3} [Fintype n] [CommRing R] [PartialOrder R] [StarRing R] [StarOrderedRing R] {M : Matrix n n R} (hM : M.PosDef) :
          M.IsHermitian
          theorem Matrix.PosDef.re_dotProduct_pos {n : Type u_2} {π•œ : Type u_4} [Fintype n] [RCLike π•œ] {M : Matrix n n π•œ} (hM : M.PosDef) {x : n β†’ π•œ} (hx : x β‰  0) :
          0 < RCLike.re (Matrix.dotProduct (star x) (M.mulVec x))
          theorem Matrix.PosDef.posSemidef {n : Type u_2} {R : Type u_3} [Fintype n] [CommRing R] [PartialOrder R] [StarRing R] [StarOrderedRing R] {M : Matrix n n R} (hM : M.PosDef) :
          M.PosSemidef
          theorem Matrix.PosDef.transpose {n : Type u_2} {R : Type u_3} [Fintype n] [CommRing R] [PartialOrder R] [StarRing R] [StarOrderedRing R] {M : Matrix n n R} (hM : M.PosDef) :
          M.transpose.PosDef
          theorem Matrix.PosDef.of_toQuadraticForm' {n : Type u_2} [Fintype n] [DecidableEq n] {M : Matrix n n ℝ} (hM : M.IsSymm) (hMq : M.toQuadraticForm'.PosDef) :
          M.PosDef
          theorem Matrix.PosDef.toQuadraticForm' {n : Type u_2} [Fintype n] [DecidableEq n] {M : Matrix n n ℝ} (hM : M.PosDef) :
          M.toQuadraticForm'.PosDef
          theorem Matrix.PosDef.eigenvalues_pos {n : Type u_2} {π•œ : Type u_4} [Fintype n] [RCLike π•œ] [DecidableEq n] {A : Matrix n n π•œ} (hA : A.PosDef) (i : n) :
          0 < β‹―.eigenvalues i

          The eigenvalues of a positive definite matrix are positive

          theorem Matrix.PosDef.det_pos {n : Type u_2} [Fintype n] [DecidableEq n] {M : Matrix n n ℝ} (hM : M.PosDef) :
          0 < M.det
          theorem QuadraticForm.posDef_of_toMatrix' {n : Type u_1} [Fintype n] [DecidableEq n] {Q : QuadraticForm ℝ (n β†’ ℝ)} (hQ : Q.toMatrix'.PosDef) :
          Q.PosDef
          theorem QuadraticForm.posDef_toMatrix' {n : Type u_1} [Fintype n] [DecidableEq n] {Q : QuadraticForm ℝ (n β†’ ℝ)} (hQ : Q.PosDef) :
          Q.toMatrix'.PosDef
          @[reducible]
          noncomputable def Matrix.NormedAddCommGroup.ofMatrix {π•œ : Type u_1} [RCLike π•œ] {n : Type u_2} [Fintype n] {M : Matrix n n π•œ} (hM : M.PosDef) :
          NormedAddCommGroup (n β†’ π•œ)

          A positive definite matrix M induces a norm β€–xβ€– = sqrt (re xα΄΄Mx).

          Equations
          Instances For
            def Matrix.InnerProductSpace.ofMatrix {π•œ : Type u_1} [RCLike π•œ] {n : Type u_2} [Fintype n] {M : Matrix n n π•œ} (hM : M.PosDef) :
            InnerProductSpace π•œ (n β†’ π•œ)

            A positive definite matrix M induces an inner product βŸͺx, y⟫ = xα΄΄My.

            Equations
            • One or more equations did not get rendered due to their size.
            Instances For