Skip to content

Commit e295847

Browse files
committed
chore(VectorBundle/Basic): minor clean-ups and polish (#26864)
Found while working on the path towards geodesics and the Levi-Civita connection.
1 parent 6d68398 commit e295847

File tree

2 files changed

+14
-8
lines changed

2 files changed

+14
-8
lines changed

β€ŽMathlib/Geometry/Manifold/VectorBundle/Basic.leanβ€Ž

Lines changed: 9 additions & 7 deletions
Original file line numberDiff line numberDiff line change
@@ -164,7 +164,8 @@ bundle at all, just that it is a fiber bundle over a charted base space.
164164

165165
namespace Bundle
166166

167-
/-- Characterization of `C^n` functions into a vector bundle. -/
167+
/-- Characterization of `C^n` functions into a vector bundle.
168+
Version at a point within a set. -/
168169
theorem contMDiffWithinAt_totalSpace {f : M β†’ TotalSpace F E} {s : Set M} {xβ‚€ : M} :
169170
ContMDiffWithinAt IM (IB.prod π“˜(π•œ, F)) n f s xβ‚€ ↔
170171
ContMDiffWithinAt IM IB n (fun x => (f x).proj) s xβ‚€ ∧
@@ -185,7 +186,7 @@ theorem contMDiffWithinAt_totalSpace {f : M β†’ TotalSpace F E} {s : Set M} {x
185186
exact hx
186187
Β· simp only [mfld_simps]
187188

188-
/-- Characterization of `C^n` functions into a vector bundle. -/
189+
/-- Characterization of `C^n` functions into a vector bundle. Version at a point. -/
189190
theorem contMDiffAt_totalSpace {f : M β†’ TotalSpace F E} {xβ‚€ : M} :
190191
ContMDiffAt IM (IB.prod π“˜(π•œ, F)) n f xβ‚€ ↔
191192
ContMDiffAt IM IB n (fun x ↦ (f x).proj) xβ‚€ ∧
@@ -213,21 +214,22 @@ theorem contMDiff_proj : ContMDiff (IB.prod π“˜(π•œ, F)) IB n (Ο€ F E) := fun
213214

214215
theorem contMDiffOn_proj {s : Set (TotalSpace F E)} :
215216
ContMDiffOn (IB.prod π“˜(π•œ, F)) IB n (Ο€ F E) s :=
216-
(Bundle.contMDiff_proj E).contMDiffOn
217+
(contMDiff_proj E).contMDiffOn
217218

218219
theorem contMDiffAt_proj {p : TotalSpace F E} : ContMDiffAt (IB.prod π“˜(π•œ, F)) IB n (Ο€ F E) p :=
219-
(Bundle.contMDiff_proj E).contMDiffAt
220+
(contMDiff_proj E).contMDiffAt
220221

221222
theorem contMDiffWithinAt_proj {s : Set (TotalSpace F E)} {p : TotalSpace F E} :
222223
ContMDiffWithinAt (IB.prod π“˜(π•œ, F)) IB n (Ο€ F E) s p :=
223-
(Bundle.contMDiffAt_proj E).contMDiffWithinAt
224+
(contMDiffAt_proj E).contMDiffWithinAt
224225

225226
variable (π•œ) [βˆ€ x, AddCommMonoid (E x)]
226227
variable [βˆ€ x, Module π•œ (E x)] [VectorBundle π•œ F E]
227228

228-
theorem contMDiff_zeroSection : ContMDiff IB (IB.prod π“˜(π•œ, F)) n (zeroSection F E) := fun x ↦ by
229+
theorem contMDiff_zeroSection : ContMDiff IB (IB.prod π“˜(π•œ, F)) n (zeroSection F E) := by
230+
intro x
229231
unfold zeroSection
230-
rw [Bundle.contMDiffAt_section]
232+
rw [contMDiffAt_section]
231233
apply (contMDiffAt_const (c := 0)).congr_of_eventuallyEq
232234
filter_upwards [(trivializationAt F E x).open_baseSet.mem_nhds
233235
(mem_baseSet_trivializationAt F E x)] with y hy

β€ŽMathlib/Geometry/Manifold/VectorBundle/MDifferentiable.leanβ€Ž

Lines changed: 5 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -32,7 +32,9 @@ variable [NontriviallyNormedField π•œ] [NormedAddCommGroup F] [NormedSpace π•œ
3232

3333
variable [TopologicalSpace B] [ChartedSpace HB B] [FiberBundle F E]
3434

35-
/-- Characterization of differentiable functions into a vector bundle. -/
35+
36+
/-- Characterization of differentiable functions into a vector bundle.
37+
Version at a point within a set -/
3638
theorem mdifferentiableWithinAt_totalSpace (f : M β†’ TotalSpace F E) {s : Set M} {xβ‚€ : M} :
3739
MDifferentiableWithinAt IM (IB.prod π“˜(π•œ, F)) f s xβ‚€ ↔
3840
MDifferentiableWithinAt IM IB (fun x => (f x).proj) s xβ‚€ ∧
@@ -54,6 +56,8 @@ theorem mdifferentiableWithinAt_totalSpace (f : M β†’ TotalSpace F E) {s : Set M
5456
exact hx
5557
Β· simp only [mfld_simps]
5658

59+
/-- Characterization of differentiable functions into a vector bundle.
60+
Version at a point -/
5761
theorem mdifferentiableAt_totalSpace (f : M β†’ TotalSpace F E) {xβ‚€ : M} :
5862
MDifferentiableAt IM (IB.prod π“˜(π•œ, F)) f xβ‚€ ↔
5963
MDifferentiableAt IM IB (fun x => (f x).proj) xβ‚€ ∧

0 commit comments

Comments
Β (0)