Skip to content
This repository has been archived by the owner on Jul 24, 2024. It is now read-only.

Commit

Permalink
fix(data/polynomial/algebra_map): fix
Browse files Browse the repository at this point in the history
  • Loading branch information
eric-wieser committed Dec 13, 2021
1 parent 4379a16 commit 9bf076a
Showing 1 changed file with 8 additions and 1 deletion.
9 changes: 8 additions & 1 deletion src/data/polynomial/algebra_map.lean
Original file line number Diff line number Diff line change
Expand Up @@ -35,6 +35,12 @@ instance algebra_of_algebra : algebra R (polynomial A) :=
function.comp_app, ring_hom.coe_comp, smul_to_finsupp, mul_to_finsupp],
exact algebra.smul_def' _ _,
end,
op_smul_def' := λ p r, begin
rcases p,
simp only [C, monomial, monomial_fun, ring_hom.coe_mk, ring_hom.to_fun_eq_coe,
function.comp_app, ring_hom.coe_comp, smul_to_finsupp, mul_to_finsupp],
exact algebra.op_smul_def' _ _,
end,
commutes' := λ r p, begin
rcases p,
simp only [C, monomial, monomial_fun, ring_hom.coe_mk, ring_hom.to_fun_eq_coe,
Expand Down Expand Up @@ -396,7 +402,8 @@ theorem not_is_unit_X_sub_C [nontrivial R] (r : R) : ¬ is_unit (X - C r) :=
end ring

lemma aeval_endomorphism {M : Type*}
[comm_ring R] [add_comm_group M] [module R M]
[comm_ring R] [add_comm_group M]
[module R M] [module Rᵐᵒᵖ M] [smul_comm_class R Rᵐᵒᵖ M] [is_central_scalar R M]
(f : M →ₗ[R] M) (v : M) (p : polynomial R) :
aeval f p v = p.sum (λ n b, b • (f ^ n) v) :=
begin
Expand Down

0 comments on commit 9bf076a

Please sign in to comment.