Skip to content

Commit

Permalink
improve comments
Browse files Browse the repository at this point in the history
  • Loading branch information
fpvandoorn authored and eric-wieser committed Oct 23, 2023
1 parent 119d99e commit f005fb5
Show file tree
Hide file tree
Showing 2 changed files with 4 additions and 4 deletions.
4 changes: 2 additions & 2 deletions src/exercises_sources/friday/manifolds.lean
Original file line number Diff line number Diff line change
Expand Up @@ -462,8 +462,7 @@ be a smooth manifold. -/
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. -/
/- Type-class inference can construct the smooth manifold structure on the tangent bundle. -/
example : smooth_manifold_with_corners (𝓑1.prod 𝓑1) (tangent_bundle 𝓑1 myℝ) :=
sorry

Expand All @@ -475,6 +474,7 @@ equal. And this would be bad.
-/
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`
-/
Expand Down
4 changes: 2 additions & 2 deletions src/solutions/friday/manifolds.lean
Original file line number Diff line number Diff line change
Expand Up @@ -515,8 +515,7 @@ be a smooth manifold. -/
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. -/
/- Type-class inference can construct the smooth manifold structure on the tangent bundle. -/
example : smooth_manifold_with_corners (𝓑1.prod 𝓑1) (tangent_bundle 𝓑1 myℝ) :=
-- sorry
by apply_instance
Expand All @@ -532,6 +531,7 @@ example : charted_space (model_prod ℝ ℝ) (tangent_bundle 𝓑1 myℝ) :=
-- sorry
by apply_instance
-- sorry

/-
The charts of any smooth vector bundle are characterized by `fiber_bundle.charted_space_chart_at`
-/
Expand Down

0 comments on commit f005fb5

Please sign in to comment.