@@ -458,7 +458,7 @@ structure vector_bundle_core (ι : Type*) :=
458
458
(mem_base_set_at : ∀ x, x ∈ base_set (index_at x))
459
459
(coord_change : ι → ι → B → (F →L[R] F))
460
460
(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))
462
462
(coord_change_comp : ∀ i j k, ∀ x ∈ (base_set i) ∩ (base_set j) ∩ (base_set k), ∀ v,
463
463
(coord_change j k x) (coord_change i j x v) = coord_change i k x v)
464
464
@@ -473,7 +473,7 @@ def trivial_vector_bundle_core (ι : Type*) [inhabited ι] :
473
473
coord_change := λ i j x, continuous_linear_map.id R F,
474
474
coord_change_self := λ i x hx v, rfl,
475
475
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 }
477
477
478
478
instance (ι : Type *) [inhabited ι] : inhabited (vector_bundle_core R B F ι) :=
479
479
⟨trivial_vector_bundle_core R B F ι⟩
@@ -483,10 +483,10 @@ namespace vector_bundle_core
483
483
variables {R B F} {ι : Type *} (Z : vector_bundle_core R B F ι)
484
484
485
485
/-- 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 :=
487
487
{ 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),
490
490
..Z }
491
491
492
492
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 :=
625
625
end ,
626
626
continuous_on_coord_change' := begin
627
627
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, _),
629
629
ext v,
630
630
exact Z.local_triv_coord_change_eq i i' hb v,
631
631
end }
0 commit comments