Skip to content

Commit

Permalink
rebuild exercises
Browse files Browse the repository at this point in the history
  • Loading branch information
eric-wieser committed Oct 23, 2023
1 parent 6b5dbb3 commit 119d99e
Showing 1 changed file with 9 additions and 3 deletions.
12 changes: 9 additions & 3 deletions src/exercises_sources/friday/manifolds.lean
Original file line number Diff line number Diff line change
Expand Up @@ -457,13 +457,14 @@ be a smooth manifold. -/
-- the type `tangent_bundle 𝓑1 myℝ` makes sense
#check tangent_bundle 𝓑1 myℝ

/- The tangent space above a point of `myℝ` is just a one-dimensional vector space (identified with `ℝ`).
/- The tangent space above a point of `myℝ` is just a one-dimensional vector space
(identified with `ℝ`).
So, one can prescribe an element of the tangent bundle as a pair (more on this below) -/
example : tangent_bundle 𝓑1 myℝ := ⟨(4 : ℝ), 0⟩

/- Construct the smooth manifold structure on the tangent bundle. Hint: the answer is a one-liner,
and this instance is not really needed. -/
instance tangent_bundle_myℝ : smooth_manifold_with_corners (𝓑1.prod 𝓑1) (tangent_bundle 𝓑1 myℝ) :=
example : smooth_manifold_with_corners (𝓑1.prod 𝓑1) (tangent_bundle 𝓑1 myℝ) :=
sorry

/-
Expand All @@ -472,7 +473,12 @@ NB: the model space for the tangent bundle to a product manifold or a tangent sp
structures with model `ℝ Γ— ℝ`, the identity one and the product one, which are not definitionally
equal. And this would be bad.
-/
#check tangent_bundle.charted_space 𝓑1 myℝ
example : charted_space (model_prod ℝ ℝ) (tangent_bundle 𝓑1 myℝ) :=
sorry
/-
The charts of any smooth vector bundle are characterized by `fiber_bundle.charted_space_chart_at`
-/
#check @fiber_bundle.charted_space_chart_at

/- A smooth map between manifolds induces a map between their tangent bundles. In `mathlib` this is
called the `tangent_map` (you might instead know it as the "differential" or "pushforward" of the
Expand Down

0 comments on commit 119d99e

Please sign in to comment.