Skip to content

Commit

Permalink
style(OneJetBundle): reflow variable block
Browse files Browse the repository at this point in the history
  • Loading branch information
grunweg committed Feb 16, 2024
1 parent 41686a8 commit 5e2a713
Showing 1 changed file with 9 additions and 8 deletions.
17 changes: 9 additions & 8 deletions SphereEversion/Global/Immersion.lean
Original file line number Diff line number Diff line change
Expand Up @@ -13,14 +13,15 @@ open scoped Manifold Topology

section General

variable {E : Type*} [NormedAddCommGroup E] [NormedSpace ℝ E] {H : Type*} [TopologicalSpace H]
(I : ModelWithCorners ℝ E H) {M : Type*} [TopologicalSpace M] [ChartedSpace H M]
[SmoothManifoldWithCorners I M] {E' : Type*} [NormedAddCommGroup E'] [NormedSpace ℝ E']
{H' : Type*} [TopologicalSpace H'] (I' : ModelWithCorners ℝ E' H') {M' : Type*}
[TopologicalSpace M'] [ChartedSpace H' M'] [SmoothManifoldWithCorners I' M'] {F : Type*}
[NormedAddCommGroup F] [NormedSpace ℝ F] {G : Type*} [TopologicalSpace G]
(J : ModelWithCorners ℝ F G) (N : Type*) [TopologicalSpace N] [ChartedSpace G N]
[SmoothManifoldWithCorners J N]
variable {E : Type*} [NormedAddCommGroup E] [NormedSpace ℝ E]
{H : Type*} [TopologicalSpace H] (I : ModelWithCorners ℝ E H) {M : Type*} [TopologicalSpace M]
[ChartedSpace H M] [SmoothManifoldWithCorners I M]
{E' : Type*} [NormedAddCommGroup E'] [NormedSpace ℝ E']
{H' : Type*} [TopologicalSpace H'] (I' : ModelWithCorners ℝ E' H')
{M' : Type*} [TopologicalSpace M'] [ChartedSpace H' M'] [SmoothManifoldWithCorners I' M']
{F : Type*} [NormedAddCommGroup F] [NormedSpace ℝ F] {G : Type*} [TopologicalSpace G]
(J : ModelWithCorners ℝ F G)
(N : Type*) [TopologicalSpace N] [ChartedSpace G N] [SmoothManifoldWithCorners J N]

local notation "TM" => TangentSpace I

Expand Down

0 comments on commit 5e2a713

Please sign in to comment.