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

Commit ed8d597

Browse files
committed
fix(data/matrix/basic): remove an accidental requirement for a matrix to be square (#8372)
1 parent fce38f1 commit ed8d597

File tree

1 file changed

+1
-1
lines changed

1 file changed

+1
-1
lines changed

src/data/matrix/basic.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -353,7 +353,7 @@ instance [has_mul α] [add_comm_monoid α] : has_mul (matrix n n α) := ⟨matri
353353
@[simp] theorem mul_eq_mul [has_mul α] [add_comm_monoid α] (M N : matrix n n α) :
354354
M * N = M ⬝ N := rfl
355355

356-
theorem mul_apply' [has_mul α] [add_comm_monoid α] {M N : matrix n n α} {i k} :
356+
theorem mul_apply' [has_mul α] [add_comm_monoid α] {M : matrix l m α} {N : matrix m n α} {i k} :
357357
(M ⬝ N) i k = dot_product (λ j, M i j) (λ j, N j k) := rfl
358358

359359
@[simp] theorem diagonal_neg [decidable_eq n] [add_group α] (d : n → α) :

0 commit comments

Comments
 (0)