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

Commit

Permalink
Update src/analysis/inner_product_space/adjoint.lean
Browse files Browse the repository at this point in the history
Co-authored-by: Frédéric Dupuis <[email protected]>
  • Loading branch information
shingtaklam1324 and dupuisf authored Sep 4, 2022
1 parent c32d8e4 commit e2f0924
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion src/analysis/inner_product_space/adjoint.lean
Original file line number Diff line number Diff line change
Expand Up @@ -103,7 +103,7 @@ linear_isometry_equiv.of_surjective

localized "postfix (name := adjoint) `†`:1000 := continuous_linear_map.adjoint" in inner_product

@[simp] lemma adjoint_apply (A : E →L[𝕜] F) (x : F) :
lemma adjoint_apply (A : E →L[𝕜] F) (x : F) :
A† x = ((to_dual 𝕜 E).symm : (normed_space.dual 𝕜 E) → E) ((to_sesq_form A) x) := rfl

/-- The fundamental property of the adjoint. -/
Expand Down

0 comments on commit e2f0924

Please sign in to comment.