Skip to content

Commit

Permalink
feat(linear_algebra/determinant): Show that the determinant is a mult…
Browse files Browse the repository at this point in the history
…ilinear map (#5142)
  • Loading branch information
eric-wieser committed Nov 30, 2020
1 parent 9f955fe commit e3a699e
Showing 1 changed file with 8 additions and 0 deletions.
8 changes: 8 additions & 0 deletions src/linear_algebra/determinant.lean
Expand Up @@ -8,6 +8,7 @@ import data.fintype.card
import group_theory.perm.sign
import algebra.algebra.basic
import tactic.ring
import linear_algebra.multilinear

universes u v w z
open equiv equiv.perm finset function
Expand Down Expand Up @@ -273,6 +274,13 @@ begin
simp [update_column_transpose, det_transpose]
end

/-- `det` is a multilinear map over the rows of the matrix -/
@[simps apply]
def det_row_multilinear : multilinear_map R (λ (i : n), n → R) R :=
{ to_fun := det,
map_add' := det_update_row_add,
map_smul' := det_update_row_smul }

@[simp] lemma det_block_diagonal {o : Type*} [fintype o] [decidable_eq o] (M : o → matrix n n R) :
(block_diagonal M).det = ∏ k, (M k).det :=
begin
Expand Down

0 comments on commit e3a699e

Please sign in to comment.