@@ -722,12 +722,12 @@ theorem mulVec_smul [Fintype n] [Monoid R] [NonUnitalNonAssocSemiring S] [Distri
722
722
723
723
@[simp]
724
724
theorem mulVec_single [Fintype n] [DecidableEq n] [NonUnitalNonAssocSemiring R] (M : Matrix m n R)
725
- (j : n) (x : R) : M *α΅₯ Pi.single j x = fun i => M i j * x :=
725
+ (j : n) (x : R) : M *α΅₯ Pi.single j x = MulOpposite.op x β’ Mα΅ j :=
726
726
funext fun _ => dotProduct_single _ _ _
727
727
728
728
@[simp]
729
729
theorem single_vecMul [Fintype m] [DecidableEq m] [NonUnitalNonAssocSemiring R] (M : Matrix m n R)
730
- (i : m) (x : R) : Pi.single i x α΅₯* M = fun j => x * M i j :=
730
+ (i : m) (x : R) : Pi.single i x α΅₯* M = x β’ M i :=
731
731
funext fun _ => single_dotProduct _ _ _
732
732
733
733
theorem mulVec_single_one [Fintype n] [DecidableEq n] [NonAssocSemiring R]
@@ -736,7 +736,7 @@ theorem mulVec_single_one [Fintype n] [DecidableEq n] [NonAssocSemiring R]
736
736
737
737
theorem single_one_vecMul [Fintype m] [DecidableEq m] [NonAssocSemiring R]
738
738
(i : m) (M : Matrix m n R) :
739
- Pi.single i 1 α΅₯* M = M i := by simp
739
+ Pi.single i 1 α΅₯* M = M i := by ext; simp
740
740
741
741
theorem diagonal_mulVec_single [Fintype n] [DecidableEq n] [NonUnitalNonAssocSemiring R] (v : n β R)
742
742
(j : n) (x : R) : diagonal v *α΅₯ Pi.single j x = Pi.single j (v j * x) := by
@@ -781,12 +781,14 @@ section NonAssocSemiring
781
781
782
782
variable [NonAssocSemiring Ξ±]
783
783
784
- theorem mulVec_one [Fintype n] (A : Matrix m n Ξ±) : A *α΅₯ 1 = fun i => β j, A i j := by
784
+ theorem mulVec_one [Fintype n] (A : Matrix m n Ξ±) : A *α΅₯ 1 = β j, Aα΅ j := by
785
785
ext; simp [mulVec, dotProduct]
786
786
787
- theorem vec_one_mul [Fintype m] (A : Matrix m n Ξ±) : 1 α΅₯* A = fun j => β i, A i j := by
787
+ theorem one_vecMul [Fintype m] (A : Matrix m n Ξ±) : 1 α΅₯* A = β i, A i := by
788
788
ext; simp [vecMul, dotProduct]
789
789
790
+ @[deprecated (since := "2025-01-26")] alias vec_one_mul := one_vecMul
791
+
790
792
variable [Fintype m] [Fintype n] [DecidableEq m]
791
793
792
794
@[simp]
0 commit comments