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

Commit 8bab60f

Browse files
committed
fix(topology/fiber_bundle/basic): rename field of fiber_bundle_core (#17679)
* Also add a `simps` attribute on one construction.
1 parent 98cdae5 commit 8bab60f

File tree

3 files changed

+11
-11
lines changed

3 files changed

+11
-11
lines changed

src/geometry/manifold/tangent_bundle.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -196,7 +196,7 @@ def to_vector_bundle_core : vector_bundle_core 𝕜 M F (atlas H M) :=
196196
{ simp only [hx1] with mfld_simps },
197197
{ simp only [hx1, hx2, hx3] with mfld_simps }
198198
end,
199-
coord_change_continuous := λ i j, begin
199+
continuous_on_coord_change := λ i j, begin
200200
refine ((Z.coord_change_continuous i j).comp' i.1.continuous_on).mono _,
201201
rintros p ⟨hp₁, hp₂⟩,
202202
refine ⟨hp₁, i.1.maps_to hp₁, _⟩,

src/topology/fiber_bundle/basic.lean

Lines changed: 4 additions & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -328,7 +328,7 @@ structure fiber_bundle_core (ι : Type*) (B : Type*) [topological_space B]
328328
(mem_base_set_at : ∀ x, x ∈ base_set (index_at x))
329329
(coord_change : ι → ι → B → F → F)
330330
(coord_change_self : ∀ i, ∀ x ∈ base_set i, ∀ v, coord_change i i x v = v)
331-
(coord_change_continuous : ∀ i j, continuous_on (λp : B × F, coord_change i j p.1 p.2)
331+
(continuous_on_coord_change : ∀ i j, continuous_on (λp : B × F, coord_change i j p.1 p.2)
332332
(((base_set i) ∩ (base_set j)) ×ˢ univ))
333333
(coord_change_comp : ∀ i j k, ∀ x ∈ (base_set i) ∩ (base_set j) ∩ (base_set k), ∀ v,
334334
(coord_change j k x) (coord_change i j x v) = coord_change i k x v)
@@ -395,9 +395,9 @@ def triv_change (i j : ι) : local_homeomorph (B × F) (B × F) :=
395395
open_target :=
396396
(is_open.inter (Z.is_open_base_set i) (Z.is_open_base_set j)).prod is_open_univ,
397397
continuous_to_fun :=
398-
continuous_on.prod continuous_fst.continuous_on (Z.coord_change_continuous i j),
398+
continuous_on.prod continuous_fst.continuous_on (Z.continuous_on_coord_change i j),
399399
continuous_inv_fun := by simpa [inter_comm]
400-
using continuous_on.prod continuous_fst.continuous_on (Z.coord_change_continuous j i) }
400+
using continuous_on.prod continuous_fst.continuous_on (Z.continuous_on_coord_change j i) }
401401

402402
@[simp, mfld_simps] lemma mem_triv_change_source (i j : ι) (p : B × F) :
403403
p ∈ (Z.triv_change i j).source ↔ p.1 ∈ Z.base_set i ∩ Z.base_set j :=
@@ -623,7 +623,7 @@ begin
623623
rw [preimage_inter, preimage_comp],
624624
by_cases (b ∈ Z.base_set i),
625625
{ have hc : continuous (λ (x : Z.fiber b), (Z.coord_change (Z.index_at b) i b) x),
626-
from (Z.coord_change_continuous (Z.index_at b) i).comp_continuous
626+
from (Z.continuous_on_coord_change (Z.index_at b) i).comp_continuous
627627
(continuous_const.prod_mk continuous_id) (λ x, ⟨⟨Z.mem_base_set_at b, h⟩, mem_univ x⟩),
628628
exact (((Z.local_triv i).open_target.inter ht).preimage (continuous.prod.mk b)).preimage hc },
629629
{ rw [(Z.local_triv i).target_eq, ←base_set_at, mk_preimage_prod_right_eq_empty h,

src/topology/vector_bundle/basic.lean

Lines changed: 6 additions & 6 deletions
Original file line numberDiff line numberDiff line change
@@ -458,7 +458,7 @@ structure vector_bundle_core (ι : Type*) :=
458458
(mem_base_set_at : ∀ x, x ∈ base_set (index_at x))
459459
(coord_change : ι → ι → B → (F →L[R] F))
460460
(coord_change_self : ∀ i, ∀ x ∈ base_set i, ∀ v, coord_change i i x v = v)
461-
(coord_change_continuous : ∀ i j, continuous_on (coord_change i j) (base_set i ∩ base_set j))
461+
(continuous_on_coord_change : ∀ i j, continuous_on (coord_change i j) (base_set i ∩ base_set j))
462462
(coord_change_comp : ∀ i j k, ∀ x ∈ (base_set i) ∩ (base_set j) ∩ (base_set k), ∀ v,
463463
(coord_change j k x) (coord_change i j x v) = coord_change i k x v)
464464

@@ -473,7 +473,7 @@ def trivial_vector_bundle_core (ι : Type*) [inhabited ι] :
473473
coord_change := λ i j x, continuous_linear_map.id R F,
474474
coord_change_self := λ i x hx v, rfl,
475475
coord_change_comp := λ i j k x hx v, rfl,
476-
coord_change_continuous := λ i j, continuous_on_const }
476+
continuous_on_coord_change := λ i j, continuous_on_const }
477477

478478
instance (ι : Type*) [inhabited ι] : inhabited (vector_bundle_core R B F ι) :=
479479
⟨trivial_vector_bundle_core R B F ι⟩
@@ -483,10 +483,10 @@ namespace vector_bundle_core
483483
variables {R B F} {ι : Type*} (Z : vector_bundle_core R B F ι)
484484

485485
/-- Natural identification to a `fiber_bundle_core`. -/
486-
def to_fiber_bundle_core : fiber_bundle_core ι B F :=
486+
@[simps (mfld_cfg)] def to_fiber_bundle_core : fiber_bundle_core ι B F :=
487487
{ coord_change := λ i j b, Z.coord_change i j b,
488-
coord_change_continuous := λ i j, is_bounded_bilinear_map_apply.continuous.comp_continuous_on
489-
((Z.coord_change_continuous i j).prod_map continuous_on_id),
488+
continuous_on_coord_change := λ i j, is_bounded_bilinear_map_apply.continuous.comp_continuous_on
489+
((Z.continuous_on_coord_change i j).prod_map continuous_on_id),
490490
..Z }
491491

492492
instance to_fiber_bundle_core_coe : has_coe (vector_bundle_core R B F ι)
@@ -625,7 +625,7 @@ instance vector_bundle : vector_bundle R F Z.fiber :=
625625
end,
626626
continuous_on_coord_change' := begin
627627
rintros _ _ ⟨i, rfl⟩ ⟨i', rfl⟩,
628-
refine (Z.coord_change_continuous i i').congr (λ b hb, _),
628+
refine (Z.continuous_on_coord_change i i').congr (λ b hb, _),
629629
ext v,
630630
exact Z.local_triv_coord_change_eq i i' hb v,
631631
end }

0 commit comments

Comments
 (0)