Skip to content

Commit

Permalink
break
Browse files Browse the repository at this point in the history
  • Loading branch information
alexjbest committed Jan 8, 2024
1 parent 7bf2295 commit efef0f9
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion test/matrix.lean
Original file line number Diff line number Diff line change
Expand Up @@ -139,7 +139,7 @@ example {α : Type _} [CommRing α] {a b c d : α} :
simp only [det_succ_row_zero, of_apply, cons_val', empty_val',
cons_val_fin_one, cons_val_zero, det_unique, Fin.default_eq_zero, submatrix_apply,
Fin.succ_zero_eq_one, cons_val_one, head_fin_const, Fin.sum_univ_succ, Fin.val_zero,
pow_zero, one_mul, Fin.zero_succAbove, head_cons, Finset.univ_unique,
pow_zero, one_mul, Fin.zero_succAbove, Finset.univ_unique,
Fin.val_succ, Fin.coe_fin_one, zero_add, pow_one, cons_val_succ, neg_mul,
Fin.succ_succAbove_zero, Finset.sum_const, Finset.card_singleton, smul_neg, one_smul]
ring
Expand Down

0 comments on commit efef0f9

Please sign in to comment.