Skip to content

Commit

Permalink
Update Mathlib/NumberTheory/NumberField/FinitePlaces.lean
Browse files Browse the repository at this point in the history
Co-authored-by: Michael Stoll <[email protected]>
  • Loading branch information
fbarroero and MichaelStollBayreuth authored Dec 3, 2024
1 parent 9b47052 commit 4a31859
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion Mathlib/NumberTheory/NumberField/FinitePlaces.lean
Original file line number Diff line number Diff line change
Expand Up @@ -227,7 +227,7 @@ theorem mulSupport_Finite {x : K} (h_x_nezero : x ≠ 0) :
map_div₀]
obtain ⟨ha, hb⟩ := h_x_nezero
simp_rw [← RingOfIntegers.coe_eq_algebraMap]
apply Set.Finite.subset (Set.Finite.union (mulSupport_Finite_int ha) (mulSupport_Finite_int hb))
apply ((mulSupport_Finite_int ha).union (mulSupport_Finite_int hb)).subset
intro w
contrapose!
intro a_1
Expand Down

0 comments on commit 4a31859

Please sign in to comment.