Skip to content

Commit

Permalink
bump to nightly-2023-07-11-13
Browse files Browse the repository at this point in the history
  • Loading branch information
leanprover-community-bot committed Jul 11, 2023
1 parent d0f0823 commit 05753d1
Show file tree
Hide file tree
Showing 3 changed files with 18 additions and 6 deletions.
12 changes: 12 additions & 0 deletions Mathbin/Geometry/Manifold/VectorBundle/Hom.lean
Expand Up @@ -45,6 +45,7 @@ variable {𝕜 B F F₁ F₂ M M₁ M₂ : Type _} {E : B → Type _} {E₁ : B

local notation "LE₁E₂" => TotalSpace (F₁ →L[𝕜] F₂) (Bundle.ContinuousLinearMap (RingHom.id 𝕜) E₁ E₂)

#print smoothOn_continuousLinearMapCoordChange /-
-- This proof is slow, especially the `simp only` and the elaboration of `h₂`.
theorem smoothOn_continuousLinearMapCoordChange [SmoothManifoldWithCorners IB B]
[SmoothVectorBundle F₁ E₁ IB] [SmoothVectorBundle F₂ E₂ IB] [MemTrivializationAtlas e₁]
Expand All @@ -66,36 +67,44 @@ theorem smoothOn_continuousLinearMapCoordChange [SmoothManifoldWithCorners IB B]
ContinuousLinearEquiv.arrowCongrSL_apply, comp_apply, Function.comp, compL_apply, flip_apply,
ContinuousLinearEquiv.symm_symm, LinearEquiv.toFun_eq_coe, ContinuousLinearMap.coe_comp']
#align smooth_on_continuous_linear_map_coord_change smoothOn_continuousLinearMapCoordChange
-/

#print hom_chart /-
theorem hom_chart (y₀ y : LE₁E₂) :
chartAt (ModelProd HB (F₁ →L[𝕜] F₂)) y₀ y =
(chartAt HB y₀.1 y.1, inCoordinates F₁ E₁ F₂ E₂ y₀.1 y.1 y₀.1 y.1 y.2) :=
by
simp_rw [FiberBundle.chartedSpace_chartAt, trans_apply, LocalHomeomorph.prod_apply,
Trivialization.coe_coe, LocalHomeomorph.refl_apply, Function.id_def, hom_trivializationAt_apply]
#align hom_chart hom_chart
-/

variable {IB}

#print contMDiffAt_hom_bundle /-
theorem contMDiffAt_hom_bundle (f : M → LE₁E₂) {x₀ : M} {n : ℕ∞} :
ContMDiffAt IM (IB.Prod 𝓘(𝕜, F₁ →L[𝕜] F₂)) n f x₀ ↔
ContMDiffAt IM IB n (fun x => (f x).1) x₀ ∧
ContMDiffAt IM 𝓘(𝕜, F₁ →L[𝕜] F₂) n
(fun x => inCoordinates F₁ E₁ F₂ E₂ (f x₀).1 (f x).1 (f x₀).1 (f x).1 (f x).2) x₀ :=
by apply cont_mdiff_at_total_space
#align cont_mdiff_at_hom_bundle contMDiffAt_hom_bundle
-/

#print smoothAt_hom_bundle /-
theorem smoothAt_hom_bundle (f : M → LE₁E₂) {x₀ : M} :
SmoothAt IM (IB.Prod 𝓘(𝕜, F₁ →L[𝕜] F₂)) f x₀ ↔
SmoothAt IM IB (fun x => (f x).1) x₀ ∧
SmoothAt IM 𝓘(𝕜, F₁ →L[𝕜] F₂)
(fun x => inCoordinates F₁ E₁ F₂ E₂ (f x₀).1 (f x).1 (f x₀).1 (f x).1 (f x).2) x₀ :=
contMDiffAt_hom_bundle f
#align smooth_at_hom_bundle smoothAt_hom_bundle
-/

variable [SmoothManifoldWithCorners IB B] [SmoothVectorBundle F₁ E₁ IB]
[SmoothVectorBundle F₂ E₂ IB]

#print Bundle.ContinuousLinearMap.vectorPrebundle.isSmooth /-
instance Bundle.ContinuousLinearMap.vectorPrebundle.isSmooth :
(Bundle.ContinuousLinearMap.vectorPrebundle (RingHom.id 𝕜) F₁ E₁ F₂ E₂).IsSmooth IB
where exists_smooth_coord_change :=
Expand All @@ -107,9 +116,12 @@ instance Bundle.ContinuousLinearMap.vectorPrebundle.isSmooth :
smoothOn_continuousLinearMapCoordChange IB,
continuous_linear_map_coord_change_apply (RingHom.id 𝕜) e₁ e₁' e₂ e₂'⟩
#align bundle.continuous_linear_map.vector_prebundle.is_smooth Bundle.ContinuousLinearMap.vectorPrebundle.isSmooth
-/

#print SmoothVectorBundle.continuousLinearMap /-
instance SmoothVectorBundle.continuousLinearMap :
SmoothVectorBundle (F₁ →L[𝕜] F₂) (Bundle.ContinuousLinearMap (RingHom.id 𝕜) E₁ E₂) IB :=
(Bundle.ContinuousLinearMap.vectorPrebundle (RingHom.id 𝕜) F₁ E₁ F₂ E₂).SmoothVectorBundle IB
#align smooth_vector_bundle.continuous_linear_map SmoothVectorBundle.continuousLinearMap
-/

8 changes: 4 additions & 4 deletions lake-manifest.json
Expand Up @@ -10,9 +10,9 @@
{"git":
{"url": "https://github.com/leanprover-community/lean3port.git",
"subDir?": null,
"rev": "ac6837f47b56ab18434422a8dfaf4673d221ec69",
"rev": "dfa812a76787276ea6c0c059f84cc20ba3c2f6cc",
"name": "lean3port",
"inputRev?": "ac6837f47b56ab18434422a8dfaf4673d221ec69"}},
"inputRev?": "dfa812a76787276ea6c0c059f84cc20ba3c2f6cc"}},
{"git":
{"url": "https://github.com/mhuisi/lean4-cli.git",
"subDir?": null,
Expand All @@ -22,9 +22,9 @@
{"git":
{"url": "https://github.com/leanprover-community/mathlib4.git",
"subDir?": null,
"rev": "51c2f54c13a4f494ea15d47ef2f91049d1a31bb0",
"rev": "fe6a0bdc715e2b574731d80a48d0d0e2a741f57f",
"name": "mathlib",
"inputRev?": "51c2f54c13a4f494ea15d47ef2f91049d1a31bb0"}},
"inputRev?": "fe6a0bdc715e2b574731d80a48d0d0e2a741f57f"}},
{"git":
{"url": "https://github.com/gebner/quote4",
"subDir?": null,
Expand Down
4 changes: 2 additions & 2 deletions lakefile.lean
Expand Up @@ -4,7 +4,7 @@ open Lake DSL System
-- Usually the `tag` will be of the form `nightly-2021-11-22`.
-- If you would like to use an artifact from a PR build,
-- it will be of the form `pr-branchname-sha`.
def tag : String := "nightly-2023-07-11-11"
def tag : String := "nightly-2023-07-11-13"
def releaseRepo : String := "leanprover-community/mathport"
def oleanTarName : String := "mathlib3-binport.tar.gz"

Expand Down Expand Up @@ -38,7 +38,7 @@ target fetchOleans (_pkg : Package) : Unit := do
untarReleaseArtifact releaseRepo tag oleanTarName libDir
return .nil

require lean3port from git "https://github.com/leanprover-community/lean3port.git"@"ac6837f47b56ab18434422a8dfaf4673d221ec69"
require lean3port from git "https://github.com/leanprover-community/lean3port.git"@"dfa812a76787276ea6c0c059f84cc20ba3c2f6cc"

@[default_target]
lean_lib Mathbin where
Expand Down

0 comments on commit 05753d1

Please sign in to comment.