Skip to content

Commit 0f6314a

Browse files
committed
feat(FieldTheory/IsAlgClosed/Basic): generalize exists_aeval_eq_zero (#31311)
from `CommRing`+`IsSimpleRing` to `CommSemiring`+`FaithfulSMul`. `Mathlib.Algebra.Algebra.IsSimpleRing` contains an instance of `FaithfulSMul` given `IsSimpleRing` if needed.
1 parent ec86c6c commit 0f6314a

File tree

2 files changed

+7
-6
lines changed

2 files changed

+7
-6
lines changed

Mathlib/FieldTheory/IsAlgClosed/Basic.lean

Lines changed: 3 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -181,9 +181,9 @@ theorem exists_aeval_eq_zero_of_injective {R : Type*} [CommSemiring R] [IsAlgClo
181181
∃ x : k, aeval x p = 0 :=
182182
exists_eval₂_eq_zero_of_injective (algebraMap R k) hinj p hp
183183

184-
theorem exists_aeval_eq_zero {R : Type*} [CommRing R] [IsSimpleRing R] [IsAlgClosed k] [Algebra R k]
185-
(p : R[X]) (hp : p.degree ≠ 0) : ∃ x : k, p.aeval x = 0 :=
186-
exists_eval₂_eq_zero _ _ hp
184+
theorem exists_aeval_eq_zero {R : Type*} [CommSemiring R] [IsAlgClosed k] [Algebra R k]
185+
[FaithfulSMul R k] (p : R[X]) (hp : p.degree ≠ 0) : ∃ x : k, p.aeval x = 0 :=
186+
exists_aeval_eq_zero_of_injective _ (FaithfulSMul.algebraMap_injective ..) _ hp
187187

188188

189189
/--

Mathlib/FieldTheory/IsSepClosed.lean

Lines changed: 4 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -171,9 +171,10 @@ theorem exists_eval₂_eq_zero {k : Type*} [CommRing k] [IsSimpleRing k] [IsSepC
171171

172172
variable (K)
173173

174-
theorem exists_aeval_eq_zero {k : Type*} [CommRing k] [IsSimpleRing k] [IsSepClosed K] [Algebra k K]
175-
(p : k[X]) (hp : p.degree ≠ 0) (hsep : p.Separable) : ∃ x : K, p.aeval x = 0 :=
176-
exists_eval₂_eq_zero _ _ hp hsep
174+
theorem exists_aeval_eq_zero {k : Type*} [CommSemiring k] [IsSepClosed K] [Algebra k K]
175+
[FaithfulSMul k K] (p : k[X]) (hp : p.degree ≠ 0) (hsep : p.Separable) :
176+
∃ x : K, p.aeval x = 0 :=
177+
exists_eval₂_eq_zero_of_injective _ (FaithfulSMul.algebraMap_injective ..) p hp hsep
177178

178179
variable (k) {K}
179180

0 commit comments

Comments
 (0)