Commit 663a7b8 1 parent be90435 commit 663a7b8 Copy full SHA for 663a7b8
File tree 1 file changed +3
-3
lines changed
Mathlib/Analysis/InnerProductSpace
1 file changed +3
-3
lines changed Original file line number Diff line number Diff line change @@ -942,7 +942,7 @@ variable {m n : Type*}
942
942
943
943
namespace Matrix
944
944
945
- variable [Fintype m] [Fintype n] [DecidableEq n]
945
+ variable [Fintype n] [DecidableEq n]
946
946
947
947
/-- `Matrix.toLin'` adapted for `EuclideanSpace 𝕜 _`. -/
948
948
def toEuclideanLin : Matrix m n 𝕜 ≃ₗ[𝕜] EuclideanSpace 𝕜 n →ₗ[𝕜] EuclideanSpace 𝕜 m :=
@@ -976,13 +976,13 @@ theorem toEuclideanLin_apply_piLp_equiv_symm (M : Matrix m n 𝕜) (v : n →
976
976
rfl
977
977
978
978
-- `Matrix.toEuclideanLin` is the same as `Matrix.toLin` applied to `PiLp.basisFun`,
979
- theorem toEuclideanLin_eq_toLin :
979
+ theorem toEuclideanLin_eq_toLin [Finite m] :
980
980
(toEuclideanLin : Matrix m n 𝕜 ≃ₗ[𝕜] _) =
981
981
Matrix.toLin (PiLp.basisFun _ _ _) (PiLp.basisFun _ _ _) :=
982
982
rfl
983
983
984
984
open EuclideanSpace in
985
- lemma toEuclideanLin_eq_toLin_orthonormal :
985
+ lemma toEuclideanLin_eq_toLin_orthonormal [Fintype m] :
986
986
toEuclideanLin = toLin (basisFun n 𝕜).toBasis (basisFun m 𝕜).toBasis :=
987
987
rfl
988
988
You can’t perform that action at this time.
0 commit comments