Skip to content

Commit eab2544

Browse files
committed
feat(SeparationQuotient): add IsTopologicalGroup instance (#23225)
Also move `nhds_mk` and deprecate it in favor of `map_mk_nhds`.
1 parent 69b18d4 commit eab2544

File tree

2 files changed

+8
-4
lines changed

2 files changed

+8
-4
lines changed

β€ŽMathlib/Topology/Algebra/SeparationQuotient/Basic.leanβ€Ž

Lines changed: 3 additions & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -92,7 +92,6 @@ instance instMul [Mul M] [ContinuousMul M] : Mul (SeparationQuotient M) where
9292
@[to_additive (attr := simp)]
9393
theorem mk_mul [Mul M] [ContinuousMul M] (a b : M) : mk (a * b) = mk a * mk b := rfl
9494

95-
9695
@[to_additive]
9796
instance instContinuousMul [Mul M] [ContinuousMul M] : ContinuousMul (SeparationQuotient M) where
9897
continuous_mul := isQuotientMap_prodMap_mk.continuous_iff.2 <| continuous_mk.comp continuous_mul
@@ -197,9 +196,9 @@ instance instGroup [Group G] [IsTopologicalGroup G] : Group (SeparationQuotient
197196
instance instCommGroup [CommGroup G] [IsTopologicalGroup G] : CommGroup (SeparationQuotient G) :=
198197
surjective_mk.commGroup mk mk_one mk_mul mk_inv mk_div mk_pow mk_zpow
199198

200-
/-- Neighborhoods in the quotient are precisely the map of neighborhoods in the prequotient. -/
201-
theorem nhds_mk (x : G) : 𝓝 (mk x) = .map mk (𝓝 x) :=
202-
le_antisymm ((SeparationQuotient.isOpenMap_mk).nhds_le x) continuous_quot_mk.continuousAt
199+
@[to_additive]
200+
instance instIsTopologicalGroup [Group G] [IsTopologicalGroup G] :
201+
IsTopologicalGroup (SeparationQuotient G) where
203202

204203
end Group
205204

β€ŽMathlib/Topology/Inseparable.leanβ€Ž

Lines changed: 5 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -605,9 +605,14 @@ theorem comap_mk_nhds_mk : comap mk (𝓝 (mk x)) = 𝓝 x :=
605605
theorem comap_mk_nhdsSet_image : comap mk (𝓝˒ (mk '' s)) = 𝓝˒ s :=
606606
(isInducing_mk.nhdsSet_eq_comap _).symm
607607

608+
/-- Push-forward of the neighborhood of a point along the projection to the separation quotient
609+
is the neighborhood of its equivalence class. -/
608610
theorem map_mk_nhds : map mk (𝓝 x) = 𝓝 (mk x) := by
609611
rw [← comap_mk_nhds_mk, map_comap_of_surjective surjective_mk]
610612

613+
@[deprecated map_mk_nhds (since := "2025-03-21")]
614+
theorem nhds_mk (x : X) : 𝓝 (mk x) = .map mk (𝓝 x) := .symm <| map_mk_nhds ..
615+
611616
theorem map_mk_nhdsSet : map mk (𝓝˒ s) = 𝓝˒ (mk '' s) := by
612617
rw [← comap_mk_nhdsSet_image, map_comap_of_surjective surjective_mk]
613618

0 commit comments

Comments
Β (0)