File tree Expand file tree Collapse file tree 3 files changed +1013
-0
lines changed Expand file tree Collapse file tree 3 files changed +1013
-0
lines changed Original file line number Diff line number Diff line change @@ -914,6 +914,7 @@ import Mathlib.Topology.Bornology.Constructions
914
914
import Mathlib.Topology.Bornology.Hom
915
915
import Mathlib.Topology.LocallyFinite
916
916
import Mathlib.Topology.NhdsSet
917
+ import Mathlib.Topology.Order
917
918
import Mathlib.Util.AtomM
918
919
import Mathlib.Util.Export
919
920
import Mathlib.Util.IncludeStr
Original file line number Diff line number Diff line change @@ -1569,6 +1569,11 @@ structure Continuous (f : α → β) : Prop where
1569
1569
is_open_preimage : ∀ s, IsOpen s → IsOpen (f ⁻¹' s)
1570
1570
#align continuous Continuous
1571
1571
1572
+ set_option quotPrecheck false in
1573
+ /-- Notation for `Continuous` with respect to a non-standard topologies. -/
1574
+ scoped [Topology] notation (name := Continuous_of) "Continuous[" t₁ ", " t₂ "]" =>
1575
+ @Continuous _ _ t₁ t₂
1576
+
1572
1577
theorem continuous_def {_ : TopologicalSpace α} {_ : TopologicalSpace β} {f : α → β} :
1573
1578
Continuous f ↔ ∀ s, IsOpen s → IsOpen (f ⁻¹' s) :=
1574
1579
⟨fun hf s hs => hf.is_open_preimage s hs, fun h => ⟨h⟩⟩
You can’t perform that action at this time.
0 commit comments