Skip to content

Commit

Permalink
feat(linear_algebra/determinant): det_units_smul and `det_is_unit_s…
Browse files Browse the repository at this point in the history
…mul` (#11206)

Add lemmas giving the determinant of a basis constructed with
`units_smul` or `is_unit_smul` with respect to the original basis.
  • Loading branch information
jsm28 committed Jan 4, 2022
1 parent 1fc7a93 commit 85784b0
Showing 1 changed file with 9 additions and 0 deletions.
9 changes: 9 additions & 0 deletions src/linear_algebra/determinant.lean
Expand Up @@ -511,3 +511,12 @@ begin
{ rw [basis.mk_coord_apply_ne hik, mul_zero, eq_comm],
exact e.det.map_eq_zero_of_eq _ (by simp [hik, function.update_apply]) hik, },
end

/-- The determinant of a basis constructed by `units_smul` is the product of the given units. -/
@[simp] lemma basis.det_units_smul (w : ι → units R) : e.det (e.units_smul w) = ∏ i, w i :=
by simp [basis.det_apply]

/-- The determinant of a basis constructed by `is_unit_smul` is the product of the given units. -/
@[simp] lemma basis.det_is_unit_smul {w : ι → R} (hw : ∀ i, is_unit (w i)) :
e.det (e.is_unit_smul hw) = ∏ i, w i :=
e.det_units_smul _

0 comments on commit 85784b0

Please sign in to comment.