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

Commit 0b51a72

Browse files
committed
feat(linear_algebra/determinant): specialize is_basis.iff_det (#7668)
After the bundled basis refactor, applying `is_basis.iff_det` in the forward direction is slightly more involved (since defining the `iff` requires an unbundled basis), so I added a lemma that does the necessary translation between "unbundled basis" and "bundled basis" for you.
1 parent 8ff2783 commit 0b51a72

File tree

1 file changed

+4
-1
lines changed

1 file changed

+4
-1
lines changed

src/linear_algebra/determinant.lean

Lines changed: 4 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -105,7 +105,7 @@ lemma basis.det_apply (v : ι → M) : e.det v = det (e.to_matrix v) := rfl
105105
lemma basis.det_self : e.det e = 1 :=
106106
by simp [e.det_apply]
107107

108-
lemma is_basis.iff_det {v : ι → M} :
108+
lemma is_basis_iff_det {v : ι → M} :
109109
linear_independent R v ∧ span R (set.range v) = ⊤ ↔ is_unit (e.det v) :=
110110
begin
111111
split,
@@ -123,3 +123,6 @@ begin
123123
rw ← this,
124124
exact ⟨v'.linear_independent, v'.span_eq⟩ },
125125
end
126+
127+
lemma basis.is_unit_det (e' : basis ι R M) : is_unit (e.det e') :=
128+
(is_basis_iff_det e).mp ⟨e'.linear_independent, e'.span_eq⟩

0 commit comments

Comments
 (0)