Skip to content
This repository was archived by the owner on Jul 24, 2024. It is now read-only.

Commit a1283d0

Browse files
committed
feat(analysis/inner_product_space/adjoint): `is_self_adjoint_iff_eq_a… (#12047)
…djoint` A self-adjoint linear map is equal to its adjoint.
1 parent 92ac8ff commit a1283d0

File tree

1 file changed

+4
-0
lines changed

1 file changed

+4
-0
lines changed

src/analysis/inner_product_space/adjoint.lean

Lines changed: 4 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -273,6 +273,10 @@ begin
273273
refine ext_inner_right_basis b (λ i, by simp only [h i, adjoint_inner_left]),
274274
end
275275

276+
lemma is_self_adjoint_iff_eq_adjoint (A : E →ₗ[𝕜] E) :
277+
is_self_adjoint A ↔ A = A.adjoint :=
278+
by rw [is_self_adjoint, ← linear_map.eq_adjoint_iff]
279+
276280
/-- `E →ₗ[𝕜] E` is a star algebra with the adjoint as the star operation. -/
277281
instance : has_star (E →ₗ[𝕜] E) := ⟨adjoint⟩
278282
instance : has_involutive_star (E →ₗ[𝕜] E) := ⟨adjoint_adjoint⟩

0 commit comments

Comments
 (0)