Skip to content

Commit af10129

Browse files
committed
feat(Algebra/Polynomial/AlgebraMap): generalize one of the ring in map_aeval_eq_aeval_map to Semiring (#14735)
... it is not needed to be commutative.
1 parent 08c93a3 commit af10129

File tree

1 file changed

+1
-1
lines changed

1 file changed

+1
-1
lines changed

Mathlib/Algebra/Polynomial/AlgebraMap.lean

+1-1
Original file line numberDiff line numberDiff line change
@@ -345,7 +345,7 @@ theorem coeff_zero_eq_aeval_zero' (p : R[X]) : algebraMap R A (p.coeff 0) = aeva
345345
simp [aeval_def]
346346
#align polynomial.coeff_zero_eq_aeval_zero' Polynomial.coeff_zero_eq_aeval_zero'
347347

348-
theorem map_aeval_eq_aeval_map {S T U : Type*} [CommSemiring S] [CommSemiring T] [Semiring U]
348+
theorem map_aeval_eq_aeval_map {S T U : Type*} [Semiring S] [CommSemiring T] [Semiring U]
349349
[Algebra R S] [Algebra T U] {φ : R →+* T} {ψ : S →+* U}
350350
(h : (algebraMap T U).comp φ = ψ.comp (algebraMap R S)) (p : R[X]) (a : S) :
351351
ψ (aeval a p) = aeval (ψ a) (p.map φ) := by

0 commit comments

Comments
 (0)