The zmod n
-algebra structure on rings whose characteristic divides n
#
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
@[protected, instance]
@[reducible]
The zmod n
-algebra structure on rings whose characteristic m
divides n
.
See note [reducible non-instances].
Equations
- zmod.algebra' R m h = {to_has_smul := {smul := λ (a : zmod n) (r : R), ↑a * r}, to_ring_hom := {to_fun := (zmod.cast_hom h R).to_fun, map_one' := _, map_mul' := _, map_zero' := _, map_add' := _}, commutes' := _, smul_def' := _}
@[reducible]
The zmod p
-algebra structure on a ring of characteristic p
. This is not an
instance since it creates a diamond with algebra.id
.
See note [reducible non-instances].
Equations
- zmod.algebra R p = zmod.algebra' R p dvd_rfl