Skip to content

Commit

Permalink
manifolds: fix lemma about tangent bundle
Browse files Browse the repository at this point in the history
  • Loading branch information
eric-wieser committed Oct 23, 2023
1 parent 9218efa commit adca715
Showing 1 changed file with 3 additions and 3 deletions.
6 changes: 3 additions & 3 deletions src/solutions/friday/manifolds.lean
Original file line number Diff line number Diff line change
Expand Up @@ -590,11 +590,11 @@ to use the library
section you_should_probably_skip_this

/- If `M` is a manifold modelled on a vector space `E`, then the underlying type for the tangent
bundle is just `Σ (x : M), tangent_space x M` (i.e., the disjoint union of the tangent spaces,
bundle is effectively `Σ (x : M), tangent_space x M` (i.e., the disjoint union of the tangent spaces,
indexed by `x` -- this is a basic object in dependent type theory). And `tangent_space x M`
is just (a copy of) `E` by definition. -/

lemma tangent_bundle_myℝ_is_prod : tangent_bundle 𝓡1 myℝ = Σ (x : myℝ), ℝ :=
lemma tangent_bundle_myℝ_is_prod : tangent_bundle 𝓡1 myℝ = bundle.total_space ℝ (λ x : myℝ, ℝ) :=
/- inline sorry -/rfl/- inline sorry -/

/- This means that you can specify a point in the tangent bundle as a pair `⟨x, v⟩`.
Expand Down Expand Up @@ -1016,7 +1016,7 @@ begin
{ rcases x with ⟨x', h'⟩,
simp at h',
simp [h'] },
{ have A : unique_mdiff_within_at 𝓡1 (Icc (0 : ℝ) 1) (⟨(x : ℝ), v⟩ : tangent_bundle 𝓡1 ℝ).fst,
{ have A : unique_mdiff_within_at 𝓡1 (Icc (0 : ℝ) 1) (⟨(x : ℝ), v⟩ : tangent_bundle 𝓡1 ℝ).proj,
{ rw unique_mdiff_within_at_iff_unique_diff_within_at,
apply unique_diff_on_Icc_zero_one _ x.2 },
change (tangent_map (𝓡∂ 1) 𝓡1 g (tangent_map_within 𝓡1 (𝓡∂ 1) f (Icc 0 1) ⟨x, v⟩)).snd = v,
Expand Down

0 comments on commit adca715

Please sign in to comment.