Skip to content

Commit

Permalink
Update Mathlib/RingTheory/Smooth/StandardSmooth.lean
Browse files Browse the repository at this point in the history
Co-authored-by: Andrew Yang <[email protected]>
  • Loading branch information
chrisflav and erdOne authored Jan 7, 2025
1 parent 2a19ed1 commit d752d6c
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion Mathlib/RingTheory/Smooth/StandardSmooth.lean
Original file line number Diff line number Diff line change
Expand Up @@ -319,7 +319,7 @@ section P

variable [Fintype P.rels] [DecidableEq P.rels]

private lemma jacobiMatrix_comp_inr_inr (i j : P.rels) :
private lemma jacobiMatrix_comp_inr_inr (i j : P.rels) :
(Q.comp P).jacobiMatrix (Sum.inr i) (Sum.inr j) =
MvPolynomial.rename Sum.inr (P.jacobiMatrix i j) := by
rw [jacobiMatrix_apply, jacobiMatrix_apply]
Expand Down

0 comments on commit d752d6c

Please sign in to comment.