Skip to content

Commit

Permalink
Rings/Z: short proof of issemigrouppreserving_mult_rng_int_mult
Browse files Browse the repository at this point in the history
  • Loading branch information
jdchristensen committed Sep 8, 2024
1 parent b70203b commit 63715eb
Showing 1 changed file with 2 additions and 17 deletions.
19 changes: 2 additions & 17 deletions theories/Algebra/Rings/Z.v
Original file line number Diff line number Diff line change
Expand Up @@ -51,23 +51,8 @@ Global Instance issemigrouppreserving_mult_rng_int_mult (R : Ring)
Proof.
intros x y.
cbn; unfold sg_op.
induction x as [|x|x].
- simpl.
by rhs nrapply rng_mult_zero_l.
- rewrite int_mul_succ_l.
rewrite grp_pow_add.
rewrite grp_pow_succ.
rhs nrapply rng_dist_r.
rewrite rng_mult_one_l.
f_ap.
- rewrite int_mul_pred_l.
rewrite grp_pow_add.
rewrite grp_pow_pred.
rhs nrapply rng_dist_r.
rewrite IHx.
f_ap.
lhs rapply (grp_homo_inv (grp_pow_homo 1)).
symmetry; apply rng_mult_negate.
lhs nrapply grp_pow_int_mul.
nrapply rng_int_mult_dist_l.
Defined.

(** [rng_int_mult R 1] is a ring homomorphism *)
Expand Down

0 comments on commit 63715eb

Please sign in to comment.