Skip to content

Commit

Permalink
anticipate Associated.lean to be fixed by #1135
Browse files Browse the repository at this point in the history
  • Loading branch information
winstonyin committed Dec 27, 2022
1 parent 594e1fe commit b12e847
Showing 1 changed file with 3 additions and 3 deletions.
6 changes: 3 additions & 3 deletions Mathlib/Algebra/Associated.lean
Expand Up @@ -838,7 +838,7 @@ instance : Preorder (Associates α) where
le_refl := dvd_refl
le_trans a b c := dvd_trans

/-- `Associates.mk` as a `MonoidHom`. -/
/-- `associates.mk` as a `monoid_hom`. -/
protected def mkMonoidHom : α →* Associates α :=
{
toFun := Associates.mk
Expand All @@ -847,9 +847,9 @@ protected def mkMonoidHom : α →* Associates α :=
#align associates.mk_monoid_hom Associates.mkMonoidHom

@[simp]
theorem mk_monoidHom_apply (a : α) : Associates.mkMonoidHom a = Associates.mk a :=
theorem mk_monoid_hom_apply (a : α) : Associates.mkMonoidHom a = Associates.mk a :=
rfl
#align associates.mk_monoid_hom_apply Associates.mk_monoidHom_apply
#align associates.mk_monoid_hom_apply Associates.mk_monoid_hom_apply

theorem associated_map_mk {f : Associates α →* α} (hinv : Function.RightInverse f Associates.mk)
(a : α) : a ~ᵤ f (Associates.mk a) :=
Expand Down

0 comments on commit b12e847

Please sign in to comment.