File tree Expand file tree Collapse file tree 1 file changed +6
-0
lines changed
Mathlib/Analysis/NormedSpace/Star Expand file tree Collapse file tree 1 file changed +6
-0
lines changed Original file line number Diff line number Diff line change @@ -184,11 +184,17 @@ lemma l2_op_norm_conjTranspose (A : Matrix m n 𝕜) : ‖Aᴴ‖ = ‖A‖ := b
184
184
toLin_conjTranspose, adjoint_toContinuousLinearMap]
185
185
exact ContinuousLinearMap.adjoint.norm_map _
186
186
187
+ lemma l2_op_nnnorm_conjTranspose (A : Matrix m n 𝕜) : ‖Aᴴ‖₊ = ‖A‖₊ :=
188
+ Subtype.ext <| l2_op_norm_conjTranspose _
189
+
187
190
lemma l2_op_norm_conjTranspose_mul_self (A : Matrix m n 𝕜) : ‖Aᴴ * A‖ = ‖A‖ * ‖A‖ := by
188
191
rw [l2_op_norm_def, toEuclideanLin_eq_toLin_orthonormal, LinearEquiv.trans_apply,
189
192
Matrix.toLin_mul (v₂ := (EuclideanSpace.basisFun m 𝕜).toBasis), toLin_conjTranspose]
190
193
exact ContinuousLinearMap.norm_adjoint_comp_self _
191
194
195
+ lemma l2_op_nnnorm_conjTranspose_mul_self (A : Matrix m n 𝕜) : ‖Aᴴ * A‖₊ = ‖A‖₊ * ‖A‖₊ :=
196
+ Subtype.ext <| l2_op_norm_conjTranspose_mul_self _
197
+
192
198
-- note: with only a type ascription in the left-hand side, Lean picks the wrong norm.
193
199
lemma l2_op_norm_mulVec (A : Matrix m n 𝕜) (x : EuclideanSpace 𝕜 n) :
194
200
‖(EuclideanSpace.equiv m 𝕜).symm <| A.mulVec x‖ ≤ ‖A‖ * ‖x‖ :=
You can’t perform that action at this time.
0 commit comments