Skip to content

Commit 663a7b8

Browse files
committed
chore(InnerProductSpace/PiL2): Fintype m -> Finite m (#15232)
1 parent be90435 commit 663a7b8

File tree

1 file changed

+3
-3
lines changed

1 file changed

+3
-3
lines changed

Mathlib/Analysis/InnerProductSpace/PiL2.lean

+3-3
Original file line numberDiff line numberDiff line change
@@ -942,7 +942,7 @@ variable {m n : Type*}
942942

943943
namespace Matrix
944944

945-
variable [Fintype m] [Fintype n] [DecidableEq n]
945+
variable [Fintype n] [DecidableEq n]
946946

947947
/-- `Matrix.toLin'` adapted for `EuclideanSpace 𝕜 _`. -/
948948
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 →
976976
rfl
977977

978978
-- `Matrix.toEuclideanLin` is the same as `Matrix.toLin` applied to `PiLp.basisFun`,
979-
theorem toEuclideanLin_eq_toLin :
979+
theorem toEuclideanLin_eq_toLin [Finite m] :
980980
(toEuclideanLin : Matrix m n 𝕜 ≃ₗ[𝕜] _) =
981981
Matrix.toLin (PiLp.basisFun _ _ _) (PiLp.basisFun _ _ _) :=
982982
rfl
983983

984984
open EuclideanSpace in
985-
lemma toEuclideanLin_eq_toLin_orthonormal :
985+
lemma toEuclideanLin_eq_toLin_orthonormal [Fintype m] :
986986
toEuclideanLin = toLin (basisFun n 𝕜).toBasis (basisFun m 𝕜).toBasis :=
987987
rfl
988988

0 commit comments

Comments
 (0)