Skip to content

Commit

Permalink
feat(algebra/squarefree): squarefree gcds of squarefree elements (#16999
Browse files Browse the repository at this point in the history
)
  • Loading branch information
alexjbest committed Oct 19, 2022
1 parent 98e8d55 commit ccbe476
Showing 1 changed file with 14 additions and 0 deletions.
14 changes: 14 additions & 0 deletions src/algebra/squarefree.lean
Original file line number Diff line number Diff line change
Expand Up @@ -82,6 +82,20 @@ lemma squarefree_of_dvd_of_squarefree [comm_monoid R]
squarefree x :=
λ a h, hsq _ (h.trans hdvd)

section squarefree_gcd_of_squarefree

variables {α : Type*} [cancel_comm_monoid_with_zero α] [gcd_monoid α]

lemma squarefree.gcd_right (a : α) {b : α} (hb : squarefree b) :
squarefree (gcd a b) :=
squarefree_of_dvd_of_squarefree (gcd_dvd_right _ _) hb

lemma squarefree.gcd_left {a : α} (b : α) (ha : squarefree a) :
squarefree (gcd a b) :=
squarefree_of_dvd_of_squarefree (gcd_dvd_left _ _) ha

end squarefree_gcd_of_squarefree

namespace multiplicity

section comm_monoid
Expand Down

0 comments on commit ccbe476

Please sign in to comment.