File tree Expand file tree Collapse file tree 2 files changed +7
-3
lines changed
Mathlib/LinearAlgebra/Matrix Expand file tree Collapse file tree 2 files changed +7
-3
lines changed Original file line number Diff line number Diff line change @@ -184,9 +184,13 @@ theorem isHermitian_mul_conjTranspose_self [Fintype n] (A : Matrix m n α) :
184184 (A * Aᴴ).IsHermitian := by rw [IsHermitian, conjTranspose_mul, conjTranspose_conjTranspose]
185185
186186/-- Note this is more general than `IsSelfAdjoint.star_mul_self` as `B` can be rectangular. -/
187- theorem isHermitian_transpose_mul_self [Fintype m] (A : Matrix m n α) : (Aᴴ * A).IsHermitian := by
187+ theorem isHermitian_conjTranspose_mul_self [Fintype m] (A : Matrix m n α) :
188+ (Aᴴ * A).IsHermitian := by
188189 rw [IsHermitian, conjTranspose_mul, conjTranspose_conjTranspose]
189190
191+ @[deprecated (since := "2025-11-10")] alias isHermitian_transpose_mul_self :=
192+ isHermitian_conjTranspose_mul_self
193+
190194/-- Note this is more general than `IsSelfAdjoint.conjugate'` as `B` can be rectangular. -/
191195theorem isHermitian_conjTranspose_mul_mul [Fintype m] {A : Matrix m m α} (B : Matrix m n α)
192196 (hA : A.IsHermitian) : (Bᴴ * A * B).IsHermitian := by
Original file line number Diff line number Diff line change @@ -203,7 +203,7 @@ theorem posSemidef_submatrix_equiv {M : Matrix n n R} (e : m ≃ n) :
203203/-- The conjugate transpose of a matrix multiplied by the matrix is positive semidefinite -/
204204theorem posSemidef_conjTranspose_mul_self [StarOrderedRing R] (A : Matrix m n R) :
205205 PosSemidef (Aᴴ * A) := by
206- refine ⟨isHermitian_transpose_mul_self _, fun x => ?_⟩
206+ refine ⟨isHermitian_conjTranspose_mul_self _, fun x => ?_⟩
207207 rw [← mulVec_mulVec, dotProduct_mulVec, vecMul_conjTranspose, star_star]
208208 exact Finset.sum_nonneg fun i _ => star_mul_self_nonneg _
209209
@@ -235,7 +235,7 @@ theorem trace_mul_conjTranspose_self_eq_zero_iff {A : Matrix m n R} :
235235end trace
236236
237237lemma eigenvalues_conjTranspose_mul_self_nonneg (A : Matrix m n 𝕜) [DecidableEq n] (i : n) :
238- 0 ≤ (isHermitian_transpose_mul_self A).eigenvalues i :=
238+ 0 ≤ (isHermitian_conjTranspose_mul_self A).eigenvalues i :=
239239 (posSemidef_conjTranspose_mul_self _).eigenvalues_nonneg _
240240
241241lemma eigenvalues_self_mul_conjTranspose_nonneg (A : Matrix m n 𝕜) [DecidableEq m] (i : m) :
You can’t perform that action at this time.
0 commit comments