Skip to content

Commit

Permalink
feat(topology/topological_fiber_bundle): a new standard construction …
Browse files Browse the repository at this point in the history
…for topological fiber bundles (#7935)

In this PR we implement a new standard construction for topological fiber bundles: namely a structure that permits to define a fiber bundle when trivializations are given as local equivalences but there is not yet a topology on the total space. The total space is hence given a topology in such a way that there is a fiber bundle structure for which the local equivalences
are also local homeomorphism and hence local trivializations.
  • Loading branch information
Nicknamen committed Jun 24, 2021
1 parent 2f27046 commit d9dcf69
Show file tree
Hide file tree
Showing 2 changed files with 266 additions and 90 deletions.
22 changes: 22 additions & 0 deletions src/topology/continuous_on.lean
Expand Up @@ -87,6 +87,22 @@ begin
exact (nhds a).sets_of_superset ((nhds a).inter_sets Hw h1) hw,
end

lemma preimage_nhds_within_coinduced' {π : α → β} {s : set β} {t : set α} {a : α}
(h : a ∈ t) (ht : is_open t)
(hs : s ∈ @nhds β (topological_space.coinduced (λ x : t, π x) subtype.topological_space) (π a)) :
π ⁻¹' s ∈ 𝓝[t] a :=
begin
letI := topological_space.coinduced (λ x : t, π x) subtype.topological_space,
rcases mem_nhds_iff.mp hs with ⟨V, hVs, V_op, mem_V⟩,
refine mem_nhds_within_iff_exists_mem_nhds_inter.mpr ⟨π ⁻¹' V, mem_nhds_iff.mpr ⟨t ∩ π ⁻¹' V,
inter_subset_right t (π ⁻¹' V), _, mem_sep h mem_V⟩, subset.trans (inter_subset_left _ _)
(preimage_mono hVs)⟩,
obtain ⟨u, hu1, hu2⟩ := is_open_induced_iff.mp (is_open_coinduced.1 V_op),
rw [preimage_comp] at hu2,
rw [set.inter_comm, ←(subtype.preimage_coe_eq_preimage_coe_iff.mp hu2)],
exact hu1.inter ht,
end

lemma mem_nhds_within_of_mem_nhds {s t : set α} {a : α} (h : s ∈ 𝓝 a) :
s ∈ 𝓝[t] a :=
mem_inf_sets_of_left h
Expand Down Expand Up @@ -151,6 +167,12 @@ theorem nhds_within_eq_of_open {a : α} {s : set α} (h₀ : a ∈ s) (h₁ : is
𝓝[s] a = 𝓝 a :=
inf_eq_left.2 $ le_principal_iff.2 $ is_open.mem_nhds h₁ h₀

lemma preimage_nhds_within_coinduced {π : α → β} {s : set β} {t : set α} {a : α}
(h : a ∈ t) (ht : is_open t)
(hs : s ∈ @nhds β (topological_space.coinduced (λ x : t, π x) subtype.topological_space) (π a)) :
π ⁻¹' s ∈ 𝓝 a :=
by { rw ←nhds_within_eq_of_open h ht, exact preimage_nhds_within_coinduced' h ht hs }

@[simp] theorem nhds_within_empty (a : α) : 𝓝[∅] a = ⊥ :=
by rw [nhds_within, principal_empty, inf_bot_eq]

Expand Down

0 comments on commit d9dcf69

Please sign in to comment.