Skip to content

Commit

Permalink
chore(ring_theory/algebra): redefine module structure of Z-algebra in…
Browse files Browse the repository at this point in the history
…stance (#1812)

This redefines the Z-algebra instance, so that the module structure is definitionally equal to the Z-module structure of any `add_comm_group`
  • Loading branch information
ChrisHughes24 authored and mergify[bot] committed Dec 18, 2019
1 parent bec46af commit 5dae5d2
Showing 1 changed file with 3 additions and 1 deletion.
4 changes: 3 additions & 1 deletion src/ring_theory/algebra.lean
Original file line number Diff line number Diff line change
Expand Up @@ -574,7 +574,9 @@ def alg_hom_int

/-- CRing ⥤ ℤ-Alg -/
instance algebra_int : algebra ℤ R :=
algebra.of_ring_hom coe $ by constructor; intros; simp
{ to_fun := coe,
commutes' := λ _ _, mul_comm _ _,
smul_def' := λ _ _, gsmul_eq_mul _ _ }

variables {R}
/-- CRing ⥤ ℤ-Alg -/
Expand Down

0 comments on commit 5dae5d2

Please sign in to comment.