File tree Expand file tree Collapse file tree 2 files changed +8
-4
lines changed
Algebra/SeparationQuotient Expand file tree Collapse file tree 2 files changed +8
-4
lines changed Original file line number Diff line number Diff line change @@ -92,7 +92,6 @@ instance instMul [Mul M] [ContinuousMul M] : Mul (SeparationQuotient M) where
9292@[to_additive (attr := simp)]
9393theorem mk_mul [Mul M] [ContinuousMul M] (a b : M) : mk (a * b) = mk a * mk b := rfl
9494
95-
9695@[to_additive]
9796instance 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
197196instance 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
204203end Group
205204
Original file line number Diff line number Diff line change @@ -605,9 +605,14 @@ theorem comap_mk_nhds_mk : comap mk (π (mk x)) = π x :=
605605theorem 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. -/
608610theorem 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+
611616theorem map_mk_nhdsSet : map mk (πΛ’ s) = πΛ’ (mk '' s) := by
612617 rw [β comap_mk_nhdsSet_image, map_comap_of_surjective surjective_mk]
613618
You canβt perform that action at this time.
0 commit comments