Skip to content

Commit 7be5fc9

Browse files
committed
feat: port Topology.Order (#1843)
1 parent 36caa8e commit 7be5fc9

File tree

3 files changed

+1013
-0
lines changed

3 files changed

+1013
-0
lines changed

Mathlib.lean

Lines changed: 1 addition & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -914,6 +914,7 @@ import Mathlib.Topology.Bornology.Constructions
914914
import Mathlib.Topology.Bornology.Hom
915915
import Mathlib.Topology.LocallyFinite
916916
import Mathlib.Topology.NhdsSet
917+
import Mathlib.Topology.Order
917918
import Mathlib.Util.AtomM
918919
import Mathlib.Util.Export
919920
import Mathlib.Util.IncludeStr

Mathlib/Topology/Basic.lean

Lines changed: 5 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -1569,6 +1569,11 @@ structure Continuous (f : α → β) : Prop where
15691569
is_open_preimage : ∀ s, IsOpen s → IsOpen (f ⁻¹' s)
15701570
#align continuous Continuous
15711571

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+
15721577
theorem continuous_def {_ : TopologicalSpace α} {_ : TopologicalSpace β} {f : α → β} :
15731578
Continuous f ↔ ∀ s, IsOpen s → IsOpen (f ⁻¹' s) :=
15741579
fun hf s hs => hf.is_open_preimage s hs, fun h => ⟨h⟩⟩

0 commit comments

Comments
 (0)