Skip to content

Commit

Permalink
chore(linear_algebra/matrix/nonsingular_inverse): replace `1 < fintyp…
Browse files Browse the repository at this point in the history
…e.card n` with `nontrivial n` (#9953)

This likely makes this a better simp lemma
  • Loading branch information
eric-wieser committed Oct 25, 2021
1 parent 0d131fe commit 87fa12a
Showing 1 changed file with 2 additions and 2 deletions.
4 changes: 2 additions & 2 deletions src/linear_algebra/matrix/nonsingular_inverse.lean
Expand Up @@ -274,10 +274,10 @@ begin
exact adjugate_subsingleton _
end

@[simp] lemma adjugate_zero (h : 1 < fintype.card n) : adjugate (0 : matrix n n α) = 0 :=
@[simp] lemma adjugate_zero [nontrivial n] : adjugate (0 : matrix n n α) = 0 :=
begin
ext i j,
obtain ⟨j', hj'⟩ : ∃ j', j' ≠ j := fintype.exists_ne_of_one_lt_card h j,
obtain ⟨j', hj'⟩ : ∃ j', j' ≠ j := exists_ne j,
apply det_eq_zero_of_column_eq_zero j',
intro j'',
simp [update_column_ne hj'],
Expand Down

0 comments on commit 87fa12a

Please sign in to comment.