File tree Expand file tree Collapse file tree 2 files changed +5
-4
lines changed Expand file tree Collapse file tree 2 files changed +5
-4
lines changed Original file line number Diff line number Diff line change @@ -779,6 +779,11 @@ theorem quot_mk_eq_mk [Monoid α] (a : α) : Quot.mk Setoid.r a = Associates.mk
779
779
rfl
780
780
#align associates.quot_mk_eq_mk Associates.quot_mk_eq_mk
781
781
782
+ @[simp]
783
+ theorem quot_out [Monoid α] (a : Associates α) : Associates.mk (Quot.out a) = a := by
784
+ rw [← quot_mk_eq_mk, Quot.out_eq]
785
+ #align associates.quot_out Associates.quot_outₓ
786
+
782
787
theorem forall_associated [Monoid α] {p : Associates α → Prop } :
783
788
(∀ a, p a) ↔ ∀ a, p (Associates.mk a) :=
784
789
Iff.intro (fun h _ => h _) fun h a => Quotient.inductionOn a h
Original file line number Diff line number Diff line change @@ -1920,10 +1920,6 @@ section
1920
1920
1921
1921
open Associates UniqueFactorizationMonoid
1922
1922
1923
- theorem Associates.quot_out {α : Type *} [CommMonoid α] (a : Associates α) :
1924
- Associates.mk (Quot.out a) = a := by rw [← quot_mk_eq_mk, Quot.out_eq]
1925
- #align associates.quot_out Associates.quot_out
1926
-
1927
1923
/-- `toGCDMonoid` constructs a GCD monoid out of a unique factorization domain. -/
1928
1924
noncomputable def UniqueFactorizationMonoid.toGCDMonoid (α : Type *) [CancelCommMonoidWithZero α]
1929
1925
[UniqueFactorizationMonoid α] [DecidableEq (Associates α)] [DecidableEq α] : GCDMonoid α where
You can’t perform that action at this time.
0 commit comments