Skip to content

Commit

Permalink
style(FieldTheory/Minpoly): rename minpoly.minpoly_lift to `minpoly…
Browse files Browse the repository at this point in the history
….lifts_algebraMap` (#22270)
  • Loading branch information
mistarro committed Feb 25, 2025
1 parent 86a0f01 commit 6d33eaf
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion Mathlib/FieldTheory/Minpoly/Field.lean
Original file line number Diff line number Diff line change
Expand Up @@ -103,7 +103,7 @@ theorem aeval_of_isScalarTower (R : Type*) {K T U : Type*} [CommRing R] [Field K

/-- If a subfield `F` of `E` contains all the coefficients of `minpoly E a`, then
`minpoly F a` maps to `minpoly E a` via `algebraMap F E`. -/
theorem minpoly_lift {F E A : Type*} [Field F] [Field E] [CommRing A]
theorem map_algebraMap {F E A : Type*} [Field F] [Field E] [CommRing A]
[Algebra F E] [Algebra E A] [Algebra F A] [IsScalarTower F E A]
{a : A} (ha : IsIntegral F a) (h : minpoly E a ∈ lifts (algebraMap F E)) :
(minpoly F a).map (algebraMap F E) = minpoly E a := by
Expand Down

0 comments on commit 6d33eaf

Please sign in to comment.