Skip to content
This repository was archived by the owner on Jul 24, 2024. It is now read-only.

Commit 15a6af2

Browse files
jcommelinmergify[bot]
authored andcommitted
feat(topology/opens): continuous.comap : opens Y → opens X (#1061)
* feat(topology/opens): continuous.comap : opens Y → opens X From the perfectoid project. * Update opens.lean
1 parent d4c7b7a commit 15a6af2

File tree

1 file changed

+15
-3
lines changed

1 file changed

+15
-3
lines changed

src/topology/opens.lean

Lines changed: 15 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -8,7 +8,7 @@ Subtype of open subsets in a topological space.
88
import topology.bases topology.subset_properties topology.constructions
99

1010
open filter lattice
11-
variables {α : Type*} [topological_space α]
11+
variables {α : Type*} {β : Type*} [topological_space α] [topological_space β]
1212

1313
namespace topological_space
1414
variable (α)
@@ -23,7 +23,6 @@ non-emptiness will be useful in metric spaces, as we will be able to put
2323
a distance (and not merely an edistance) on this space. -/
2424
def nonempty_compacts := {s : set α // s ≠ ∅ ∧ compact s}
2525

26-
2726
section nonempty_compacts
2827
open topological_space set
2928
variable {α}
@@ -50,7 +49,6 @@ instance : has_subset (opens α) :=
5049
instance : has_mem α (opens α) :=
5150
{ mem := λ a U, a ∈ U.val }
5251

53-
5452
@[extensionality] lemma ext {U V : opens α} (h : U.val = V.val) : U = V := subtype.ext.mpr h
5553

5654
instance : partial_order (opens α) := subtype.partial_order _
@@ -164,3 +162,17 @@ end
164162
end opens
165163

166164
end topological_space
165+
166+
namespace continuous
167+
open topological_space
168+
169+
def comap {f : α → β} (hf : continuous f) (V : opens β) : opens α :=
170+
⟨f ⁻¹' V.1, hf V.1 V.2
171+
172+
@[simp] lemma comap_id (U : opens α) : (continuous_id).comap U = U := by { ext, refl }
173+
174+
lemma comap_mono {f : α → β} (hf : continuous f) {V W : opens β} (hVW : V ⊆ W) :
175+
hf.comap V ⊆ hf.comap W :=
176+
λ _ h, hVW h
177+
178+
end continuous

0 commit comments

Comments
 (0)