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

Commit 2910c07

Browse files
committed
fix(data/zmod/algebra): fix
1 parent 9bf076a commit 2910c07

File tree

1 file changed

+2
-0
lines changed

1 file changed

+2
-0
lines changed

src/data/zmod/algebra.lean

Lines changed: 2 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -21,6 +21,7 @@ variables {n : ℕ} (m : ℕ) [char_p R m]
2121
/-- The `zmod n`-algebra structure on rings whose characteristic `m` divides `n` -/
2222
def algebra' (h : m ∣ n) : algebra (zmod n) R :=
2323
{ smul := λ a r, a * r,
24+
to_opposite_has_scalar := { smul := λ a r, r * a },
2425
commutes' := λ a r, show (a * r : R) = r * a,
2526
begin
2627
rcases zmod.int_cast_surjective a with ⟨k, rfl⟩,
@@ -29,6 +30,7 @@ def algebra' (h : m ∣ n) : algebra (zmod n) R :=
2930
exact commute.cast_int_left r k,
3031
end,
3132
smul_def' := λ a r, rfl,
33+
op_smul_def' := λ r a, rfl,
3234
.. zmod.cast_hom h R }
3335

3436
end

0 commit comments

Comments
 (0)