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

Commit 9bf076a

Browse files
committed
fix(data/polynomial/algebra_map): fix
1 parent 4379a16 commit 9bf076a

File tree

1 file changed

+8
-1
lines changed

1 file changed

+8
-1
lines changed

src/data/polynomial/algebra_map.lean

Lines changed: 8 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -35,6 +35,12 @@ instance algebra_of_algebra : algebra R (polynomial A) :=
3535
function.comp_app, ring_hom.coe_comp, smul_to_finsupp, mul_to_finsupp],
3636
exact algebra.smul_def' _ _,
3737
end,
38+
op_smul_def' := λ p r, begin
39+
rcases p,
40+
simp only [C, monomial, monomial_fun, ring_hom.coe_mk, ring_hom.to_fun_eq_coe,
41+
function.comp_app, ring_hom.coe_comp, smul_to_finsupp, mul_to_finsupp],
42+
exact algebra.op_smul_def' _ _,
43+
end,
3844
commutes' := λ r p, begin
3945
rcases p,
4046
simp only [C, monomial, monomial_fun, ring_hom.coe_mk, ring_hom.to_fun_eq_coe,
@@ -396,7 +402,8 @@ theorem not_is_unit_X_sub_C [nontrivial R] (r : R) : ¬ is_unit (X - C r) :=
396402
end ring
397403

398404
lemma aeval_endomorphism {M : Type*}
399-
[comm_ring R] [add_comm_group M] [module R M]
405+
[comm_ring R] [add_comm_group M]
406+
[module R M] [module Rᵐᵒᵖ M] [smul_comm_class R Rᵐᵒᵖ M] [is_central_scalar R M]
400407
(f : M →ₗ[R] M) (v : M) (p : polynomial R) :
401408
aeval f p v = p.sum (λ n b, b • (f ^ n) v) :=
402409
begin

0 commit comments

Comments
 (0)