We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
map_aeval_eq_aeval_map
Semiring
1 parent 08c93a3 commit af10129Copy full SHA for af10129
Mathlib/Algebra/Polynomial/AlgebraMap.lean
@@ -345,7 +345,7 @@ theorem coeff_zero_eq_aeval_zero' (p : R[X]) : algebraMap R A (p.coeff 0) = aeva
345
simp [aeval_def]
346
#align polynomial.coeff_zero_eq_aeval_zero' Polynomial.coeff_zero_eq_aeval_zero'
347
348
-theorem map_aeval_eq_aeval_map {S T U : Type*} [CommSemiring S] [CommSemiring T] [Semiring U]
+theorem map_aeval_eq_aeval_map {S T U : Type*} [Semiring S] [CommSemiring T] [Semiring U]
349
[Algebra R S] [Algebra T U] {φ : R →+* T} {ψ : S →+* U}
350
(h : (algebraMap T U).comp φ = ψ.comp (algebraMap R S)) (p : R[X]) (a : S) :
351
ψ (aeval a p) = aeval (ψ a) (p.map φ) := by
0 commit comments