Skip to content

Commit

Permalink
name change
Browse files Browse the repository at this point in the history
Co-authored-by: Yaël Dillies <[email protected]>
  • Loading branch information
hannahfechtner and YaelDillies authored Oct 31, 2024
1 parent d5bd1c7 commit 10bdf06
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion Mathlib/GroupTheory/Congruence/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -74,7 +74,7 @@ theorem congr_mk {c d : Con M} (h : c = d) (a : M) :
Con.congr h (a : c.Quotient) = (a : d.Quotient) := rfl

@[to_additive]
theorem conGen_le_comap {M N : Type*} [Mul M] [Mul N] (f : M → N)
theorem le_comap_conGen {M N : Type*} [Mul M] [Mul N] (f : M → N)
(H : ∀ (x y : M), f (x * y) = f x * f y) (rel : N → N → Prop) :
conGen (fun x y ↦ rel (f x) (f y)) ≤ Con.comap f H (conGen rel) := by
intro x y h
Expand Down

0 comments on commit 10bdf06

Please sign in to comment.