Skip to content

Commit

Permalink
feat(data/int/cast): monoid_hom.ext_int (#3587)
Browse files Browse the repository at this point in the history
Co-authored-by: Chris Hughes <33847686+ChrisHughes24@users.noreply.github.com>
  • Loading branch information
ChrisHughes24 and ChrisHughes24 committed Jul 27, 2020
1 parent 864a22a commit 7556353
Showing 1 changed file with 14 additions and 0 deletions.
14 changes: 14 additions & 0 deletions src/data/int/cast.lean
Original file line number Diff line number Diff line change
Expand Up @@ -184,6 +184,20 @@ ext_iff.1 (f.eq_int_cast_hom h1)

end add_monoid_hom

namespace monoid_hom
variables {M : Type*} [monoid M]
open multiplicative

theorem ext_int {f g : multiplicative ℤ →* M}
(h1 : f (of_add 1) = g (of_add 1)) : f = g :=
begin
ext,
exact add_monoid_hom.ext_iff.1
(@add_monoid_hom.ext_int _ _ f.to_additive g.to_additive h1) _,
end

end monoid_hom

namespace ring_hom

variables {α : Type*} {β : Type*} [ring α] [ring β]
Expand Down

0 comments on commit 7556353

Please sign in to comment.