Skip to content

Commit bfe06a7

Browse files
winstonyinChrisHughes24hrmacbeth
committed
feat: port Algebra.GCDMonoid.Basic (#1135)
Co-authored-by: Chris Hughes <33847686+ChrisHughes24@users.noreply.github.com> Co-authored-by: Heather Macbeth <25316162+hrmacbeth@users.noreply.github.com>
1 parent 21c7a6b commit bfe06a7

File tree

6 files changed

+1443
-5
lines changed

6 files changed

+1443
-5
lines changed

Mathlib.lean

Lines changed: 1 addition & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -12,6 +12,7 @@ import Mathlib.Algebra.Field.Basic
1212
import Mathlib.Algebra.Field.Defs
1313
import Mathlib.Algebra.Field.Opposite
1414
import Mathlib.Algebra.Field.Power
15+
import Mathlib.Algebra.GCDMonoid.Basic
1516
import Mathlib.Algebra.Group.Basic
1617
import Mathlib.Algebra.Group.Commutator
1718
import Mathlib.Algebra.Group.Commute

Mathlib/Algebra/Associated.lean

Lines changed: 3 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -838,7 +838,7 @@ instance : Preorder (Associates α) where
838838
le_refl := dvd_refl
839839
le_trans a b c := dvd_trans
840840

841-
/-- `associates.mk` as a `monoid_hom`. -/
841+
/-- `Associates.mk` as a `MonoidHom`. -/
842842
protected def mkMonoidHom : α →* Associates α :=
843843
{
844844
toFun := Associates.mk
@@ -847,9 +847,9 @@ protected def mkMonoidHom : α →* Associates α :=
847847
#align associates.mk_monoid_hom Associates.mkMonoidHom
848848

849849
@[simp]
850-
theorem mk_monoid_hom_apply (a : α) : Associates.mkMonoidHom a = Associates.mk a :=
850+
theorem mk_monoidHom_apply (a : α) : Associates.mkMonoidHom a = Associates.mk a :=
851851
rfl
852-
#align associates.mk_monoid_hom_apply Associates.mk_monoid_hom_apply
852+
#align associates.mk_monoid_hom_apply Associates.mk_monoidHom_apply
853853

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

Mathlib/Algebra/Divisibility/Basic.lean

Lines changed: 3 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -74,6 +74,9 @@ alias dvd_trans ← Dvd.dvd.trans
7474
instance : IsTrans α (· ∣ ·) :=
7575
fun _ _ _ => dvd_trans⟩
7676

77+
/-- Transitivity of `|` for use in `calc` blocks -/
78+
instance : @Trans α α α Dvd.dvd Dvd.dvd Dvd.dvd := ⟨dvd_trans⟩
79+
7780
@[simp]
7881
theorem dvd_mul_right (a b : α) : a ∣ a * b :=
7982
Dvd.intro b rfl

0 commit comments

Comments
 (0)