Skip to content

Commit

Permalink
feat(linear_algebra/determinant): basis.det_ne_zero (#10126)
Browse files Browse the repository at this point in the history
Add the trivial lemma that the determinant with respect to a basis is
not the zero map (if the ring is nontrivial).
  • Loading branch information
jsm28 committed Nov 2, 2021
1 parent 86ed02f commit 123db5e
Showing 1 changed file with 4 additions and 0 deletions.
4 changes: 4 additions & 0 deletions src/linear_algebra/determinant.lean
Expand Up @@ -342,6 +342,10 @@ lemma basis.det_apply (v : ι → M) : e.det v = det (e.to_matrix v) := rfl
lemma basis.det_self : e.det e = 1 :=
by simp [e.det_apply]

/-- `basis.det` is not the zero map. -/
lemma basis.det_ne_zero [nontrivial R] : e.det ≠ 0 :=
λ h, by simpa [h] using e.det_self

lemma is_basis_iff_det {v : ι → M} :
linear_independent R v ∧ span R (set.range v) = ⊤ ↔ is_unit (e.det v) :=
begin
Expand Down

0 comments on commit 123db5e

Please sign in to comment.