File tree Expand file tree Collapse file tree 2 files changed +2
-2
lines changed
Mathlib/Algebra/GCDMonoid Expand file tree Collapse file tree 2 files changed +2
-2
lines changed Original file line number Diff line number Diff line change @@ -173,7 +173,7 @@ theorem gcd_image [DecidableEq β] {g : γ → β} (s : Finset γ) :
173
173
theorem gcd_eq_gcd_image [DecidableEq α] : s.gcd f = (s.image f).gcd id :=
174
174
Eq.symm <| gcd_image _
175
175
176
- theorem gcd_eq_zero_iff : s.gcd f = 0 ↔ ∀ x : β, x ∈ s → f x = 0 := by
176
+ theorem gcd_eq_zero_iff : s.gcd f = 0 ↔ ∀ x ∈ s, f x = 0 := by
177
177
rw [gcd_def, Multiset.gcd_eq_zero_iff]
178
178
constructor <;> intro h
179
179
· intro b bs
Original file line number Diff line number Diff line change @@ -140,7 +140,7 @@ theorem gcd_mono {s₁ s₂ : Multiset α} (h : s₁ ⊆ s₂) : s₂.gcd ∣ s
140
140
theorem normalize_gcd (s : Multiset α) : normalize s.gcd = s.gcd :=
141
141
Multiset.induction_on s (by simp) fun a s _ ↦ by simp
142
142
143
- theorem gcd_eq_zero_iff (s : Multiset α) : s.gcd = 0 ↔ ∀ x : α, x ∈ s → x = 0 := by
143
+ theorem gcd_eq_zero_iff (s : Multiset α) : s.gcd = 0 ↔ ∀ x ∈ s, x = 0 := by
144
144
constructor
145
145
· intro h x hx
146
146
apply eq_zero_of_zero_dvd
You can’t perform that action at this time.
0 commit comments