Skip to content

Commit

Permalink
fix @Basis.mk
Browse files Browse the repository at this point in the history
  • Loading branch information
alreadydone committed Jan 5, 2025
1 parent 51ffcb5 commit 4a0e6a9
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion Mathlib/RingTheory/AdjoinRoot.lean
Original file line number Diff line number Diff line change
Expand Up @@ -506,7 +506,7 @@ def powerBasisAux (hf : f ≠ 0) : Basis (Fin f.natDegree) K (AdjoinRoot f) := b
rw [natDegree_mul hf, natDegree_C, add_zero]
· rwa [Ne, C_eq_zero, inv_eq_zero, leadingCoeff_eq_zero]
have minpoly_eq : minpoly K (root f) = f' := minpoly_root hf
apply @Basis.mk _ _ _ fun i : Fin f.natDegree => root f ^ i.val
apply Basis.mk (v := fun i : Fin f.natDegree root f ^ i.val)
· rw [← deg_f', ← minpoly_eq]
exact linearIndependent_pow (root f)
· rintro y -
Expand Down

0 comments on commit 4a0e6a9

Please sign in to comment.