Skip to content

Commit

Permalink
fix(TopologicalSpace/Basic): restore curly braces in continuous_def (
Browse files Browse the repository at this point in the history
…#10110)

These were placed on purpose; reverting them caused breakage downstream.



Co-authored-by: grunweg <grunweg@posteo.de>
Co-authored-by: Yury G. Kudryashov <urkud@urkud.name>
  • Loading branch information
3 people committed Feb 16, 2024
1 parent e554fa5 commit a2f4883
Showing 1 changed file with 6 additions and 3 deletions.
9 changes: 6 additions & 3 deletions Mathlib/Topology/Basic.lean
Expand Up @@ -1499,12 +1499,15 @@ variable {X Y Z : Type*} [TopologicalSpace X] [TopologicalSpace Y] [TopologicalS

open TopologicalSpace

variable {f : X → Y} {s : Set X} {x : X} {y : Y}

theorem continuous_def : Continuous f ↔ ∀ s, IsOpen s → IsOpen (f ⁻¹' s) :=
-- The curly braces are intentional, so this definition works well with simp
-- when topologies are not those provided by instances.
theorem continuous_def {_ : TopologicalSpace X} {_ : TopologicalSpace Y} {f : X → Y} :
Continuous f ↔ ∀ s, IsOpen s → IsOpen (f ⁻¹' s) :=
fun hf => hf.1, fun h => ⟨h⟩⟩
#align continuous_def continuous_def

variable {f : X → Y} {s : Set X} {x : X} {y : Y}

theorem IsOpen.preimage (hf : Continuous f) {t : Set Y} (h : IsOpen t) :
IsOpen (f ⁻¹' t) :=
hf.isOpen_preimage t h
Expand Down

0 comments on commit a2f4883

Please sign in to comment.