We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
There was an error while loading. Please reload this page.
1 parent 6034096 commit c3b95a7Copy full SHA for c3b95a7
Mathlib/LinearAlgebra/Matrix/PosDef.lean
@@ -171,6 +171,11 @@ lemma eigenvalues_nonneg [DecidableEq n] {A : Matrix n n 𝕜}
171
(hA : Matrix.PosSemidef A) (i : n) : 0 ≤ hA.1.eigenvalues i :=
172
(hA.re_dotProduct_nonneg _).trans_eq (hA.1.eigenvalues_eq _).symm
173
174
+theorem det_nonneg [DecidableEq n] {M : Matrix n n 𝕜} (hM : M.PosSemidef) :
175
+ 0 ≤ M.det := by
176
+ rw [hM.isHermitian.det_eq_prod_eigenvalues]
177
+ exact Finset.prod_nonneg fun i _ ↦ by simpa using hM.eigenvalues_nonneg i
178
+
179
section sqrt
180
181
variable [DecidableEq n] {A : Matrix n n 𝕜} (hA : PosSemidef A)
0 commit comments