Skip to content

Commit

Permalink
chore(ring_theory/ideal/operations): generalize typeclass in map_map …
Browse files Browse the repository at this point in the history
…and comap_comap (#10077)

Split from #10024 which is hitting timeouts somewhere more irritating.
  • Loading branch information
eric-wieser committed Oct 31, 2021
1 parent 233eb66 commit 106dc57
Showing 1 changed file with 4 additions and 4 deletions.
8 changes: 4 additions & 4 deletions src/ring_theory/ideal/operations.lean
Original file line number Diff line number Diff line change
Expand Up @@ -787,11 +787,11 @@ ideal.ext $ λ _, iff.rfl
@[simp] lemma map_id : I.map (ring_hom.id R) = I :=
(gc_map_comap (ring_hom.id R)).l_unique galois_connection.id comap_id

lemma comap_comap {T : Type*} [ring T] {I : ideal T} (f : R →+* S)
(g : S →+*T) : (I.comap g).comap f = I.comap (g.comp f) := rfl
lemma comap_comap {T : Type*} [semiring T] {I : ideal T} (f : R →+* S)
(g : S →+* T) : (I.comap g).comap f = I.comap (g.comp f) := rfl

lemma map_map {T : Type*} [ring T] {I : ideal R} (f : R →+* S)
(g : S →+*T) : (I.map f).map g = I.map (g.comp f) :=
lemma map_map {T : Type*} [semiring T] {I : ideal R} (f : R →+* S)
(g : S →+* T) : (I.map f).map g = I.map (g.comp f) :=
((gc_map_comap f).compose (gc_map_comap g)).l_unique
(gc_map_comap (g.comp f)) (λ _, comap_comap _ _)

Expand Down

0 comments on commit 106dc57

Please sign in to comment.