geometry.manifold.derivation_bundle
โท
Mathlib.Geometry.Manifold.DerivationBundle
The following section lists changes to this file in mathlib3 and mathlib4 that occured after the initial port. Most recent changes are shown first. Hovering over a commit will show all commits associated with the same mathlib3 commit.
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(no changes)
(last sync)
mathlib commit https://github.com/leanprover-community/mathlib/commit/65a1391a0106c9204fe45bc73a039f056558cb83
@@ -57,10 +57,10 @@ variable {๐ M}
namespace PointedSmoothMap
-#print PointedSmoothMap.instDFunLike /-
-instance instDFunLike {x : M} : DFunLike C^โโฎI, M; ๐โฏโจxโฉ M fun _ => ๐ :=
- ContMDiffMap.instDFunLike
-#align pointed_smooth_map.fun_like PointedSmoothMap.instDFunLike
+#print PointedSmoothMap.instFunLike /-
+instance instFunLike {x : M} : DFunLike C^โโฎI, M; ๐โฏโจxโฉ M fun _ => ๐ :=
+ ContMDiffMap.instFunLike
+#align pointed_smooth_map.fun_like PointedSmoothMap.instFunLike
-/
instance {x : M} : CommRing C^โโฎI, M; ๐โฏโจxโฉ :=
mathlib commit https://github.com/leanprover-community/mathlib/commit/65a1391a0106c9204fe45bc73a039f056558cb83
@@ -57,10 +57,10 @@ variable {๐ M}
namespace PointedSmoothMap
-#print PointedSmoothMap.funLike /-
-instance funLike {x : M} : FunLike C^โโฎI, M; ๐โฏโจxโฉ M fun _ => ๐ :=
- ContMDiffMap.funLike
-#align pointed_smooth_map.fun_like PointedSmoothMap.funLike
+#print PointedSmoothMap.instDFunLike /-
+instance instDFunLike {x : M} : DFunLike C^โโฎI, M; ๐โฏโจxโฉ M fun _ => ๐ :=
+ ContMDiffMap.instDFunLike
+#align pointed_smooth_map.fun_like PointedSmoothMap.instDFunLike
-/
instance {x : M} : CommRing C^โโฎI, M; ๐โฏโจxโฉ :=
mathlib commit https://github.com/leanprover-community/mathlib/commit/ce64cd319bb6b3e82f31c2d38e79080d377be451
@@ -3,8 +3,8 @@ Copyright ยฉ 2020 Nicolรฒ Cavalleri. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Nicolรฒ Cavalleri
-/
-import Mathbin.Geometry.Manifold.Algebra.SmoothFunctions
-import Mathbin.RingTheory.Derivation.Basic
+import Geometry.Manifold.Algebra.SmoothFunctions
+import RingTheory.Derivation.Basic
#align_import geometry.manifold.derivation_bundle from "leanprover-community/mathlib"@"728ef9dbb281241906f25cbeb30f90d83e0bb451"
mathlib commit https://github.com/leanprover-community/mathlib/commit/8ea5598db6caeddde6cb734aa179cc2408dbd345
@@ -2,15 +2,12 @@
Copyright ยฉ 2020 Nicolรฒ Cavalleri. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Nicolรฒ Cavalleri
-
-! This file was ported from Lean 3 source module geometry.manifold.derivation_bundle
-! leanprover-community/mathlib commit 728ef9dbb281241906f25cbeb30f90d83e0bb451
-! Please do not edit these lines, except to modify the commit id
-! if you have ported upstream changes.
-/
import Mathbin.Geometry.Manifold.Algebra.SmoothFunctions
import Mathbin.RingTheory.Derivation.Basic
+#align_import geometry.manifold.derivation_bundle from "leanprover-community/mathlib"@"728ef9dbb281241906f25cbeb30f90d83e0bb451"
+
/-!
# Derivation bundle
mathlib commit https://github.com/leanprover-community/mathlib/commit/728ef9dbb281241906f25cbeb30f90d83e0bb451
@@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Nicolรฒ Cavalleri
! This file was ported from Lean 3 source module geometry.manifold.derivation_bundle
-! leanprover-community/mathlib commit 86c29aefdba50b3f33e86e52e3b2f51a0d8f0282
+! leanprover-community/mathlib commit 728ef9dbb281241906f25cbeb30f90d83e0bb451
! Please do not edit these lines, except to modify the commit id
! if you have ported upstream changes.
-/
@@ -15,6 +15,9 @@ import Mathbin.RingTheory.Derivation.Basic
# Derivation bundle
+> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
+> Any changes to this file require a corresponding PR to mathlib4.
+
In this file we define the derivations at a point of a manifold on the algebra of smooth fuctions.
Moreover, we define the differential of a function in terms of derivations.
mathlib commit https://github.com/leanprover-community/mathlib/commit/9240e8be927a0955b9a82c6c85ef499ee3a626b8
@@ -31,19 +31,25 @@ variable (๐ : Type _) [NontriviallyNormedField ๐] {E : Type _} [NormedAddC
open scoped Manifold
+#print smoothFunctionsAlgebra /-
-- the following two instances prevent poorly understood type class inference timeout problems
instance smoothFunctionsAlgebra : Algebra ๐ C^โโฎI, M; ๐โฏ := by infer_instance
#align smooth_functions_algebra smoothFunctionsAlgebra
+-/
+#print smooth_functions_tower /-
instance smooth_functions_tower : IsScalarTower ๐ C^โโฎI, M; ๐โฏ C^โโฎI, M; ๐โฏ := by infer_instance
#align smooth_functions_tower smooth_functions_tower
+-/
+#print PointedSmoothMap /-
/-- Type synonym, introduced to put a different `has_smul` action on `C^nโฎI, M; ๐โฏ`
which is defined as `f โข r = f(x) * r`. -/
@[nolint unused_arguments]
def PointedSmoothMap (x : M) :=
C^nโฎI, M; ๐โฏ
#align pointed_smooth_map PointedSmoothMap
+-/
scoped[Derivation] notation "C^" n "โฎ" I ", " M "; " ๐ "โฏโจ" x "โฉ" => PointedSmoothMap ๐ I M n x
@@ -51,9 +57,11 @@ variable {๐ M}
namespace PointedSmoothMap
+#print PointedSmoothMap.funLike /-
instance funLike {x : M} : FunLike C^โโฎI, M; ๐โฏโจxโฉ M fun _ => ๐ :=
ContMDiffMap.funLike
#align pointed_smooth_map.fun_like PointedSmoothMap.funLike
+-/
instance {x : M} : CommRing C^โโฎI, M; ๐โฏโจxโฉ :=
SmoothMap.commRing
@@ -72,19 +80,25 @@ instance {x : M} : IsScalarTower ๐ C^โโฎI, M; ๐โฏโจxโฉ C^โโฎI, M;
variable {I}
+#print PointedSmoothMap.evalAlgebra /-
/-- `smooth_map.eval_ring_hom` gives rise to an algebra structure of `C^โโฎI, M; ๐โฏ` on `๐`. -/
instance evalAlgebra {x : M} : Algebra C^โโฎI, M; ๐โฏโจxโฉ ๐ :=
(SmoothMap.evalRingHom x : C^โโฎI, M; ๐โฏโจxโฉ โ+* ๐).toAlgebra
#align pointed_smooth_map.eval_algebra PointedSmoothMap.evalAlgebra
+-/
+#print PointedSmoothMap.eval /-
/-- With the `eval_algebra` algebra structure evaluation is actually an algebra morphism. -/
def eval (x : M) : C^โโฎI, M; ๐โฏ โโ[C^โโฎI, M; ๐โฏโจxโฉ] ๐ :=
Algebra.ofId C^โโฎI, M; ๐โฏโจxโฉ ๐
#align pointed_smooth_map.eval PointedSmoothMap.eval
+-/
+#print PointedSmoothMap.smul_def /-
theorem smul_def (x : M) (f : C^โโฎI, M; ๐โฏโจxโฉ) (k : ๐) : f โข k = f x * k :=
rfl
#align pointed_smooth_map.smul_def PointedSmoothMap.smul_def
+-/
instance (x : M) : IsScalarTower ๐ C^โโฎI, M; ๐โฏโจxโฉ ๐
where smul_assoc k f h := by
@@ -94,35 +108,43 @@ end PointedSmoothMap
open scoped Derivation
+#print PointDerivation /-
/-- The derivations at a point of a manifold. Some regard this as a possible definition of the
tangent space -/
@[reducible]
def PointDerivation (x : M) :=
Derivation ๐ C^โโฎI, M; ๐โฏโจxโฉ ๐
#align point_derivation PointDerivation
+-/
section
variable (I) {M} (X Y : Derivation ๐ C^โโฎI, M; ๐โฏ C^โโฎI, M; ๐โฏ) (f g : C^โโฎI, M; ๐โฏ) (r : ๐)
+#print SmoothFunction.evalAt /-
/-- Evaluation at a point gives rise to a `C^โโฎI, M; ๐โฏ`-linear map between `C^โโฎI, M; ๐โฏ` and `๐`.
-/
def SmoothFunction.evalAt (x : M) : C^โโฎI, M; ๐โฏ โโ[C^โโฎI, M; ๐โฏโจxโฉ] ๐ :=
(PointedSmoothMap.eval x).toLinearMap
#align smooth_function.eval_at SmoothFunction.evalAt
+-/
namespace Derivation
variable {I}
+#print Derivation.evalAt /-
/-- The evaluation at a point as a linear map. -/
def evalAt (x : M) : Derivation ๐ C^โโฎI, M; ๐โฏ C^โโฎI, M; ๐โฏ โโ[๐] PointDerivation I x :=
(SmoothFunction.evalAt I x).compDer
#align derivation.eval_at Derivation.evalAt
+-/
+#print Derivation.evalAt_apply /-
theorem evalAt_apply (x : M) : evalAt x X f = (X f) x :=
rfl
#align derivation.eval_at_apply Derivation.evalAt_apply
+-/
end Derivation
@@ -130,6 +152,7 @@ variable {I} {E' : Type _} [NormedAddCommGroup E'] [NormedSpace ๐ E'] {H' : T
[TopologicalSpace H'] {I' : ModelWithCorners ๐ E' H'} {M' : Type _} [TopologicalSpace M']
[ChartedSpace H' M']
+#print hfdifferential /-
/-- The heterogeneous differential as a linear map. Instead of taking a function as an argument this
differential takes `h : f x = y`. It is particularly handy to deal with situations where the points
on where it has to be evaluated are equal but not definitionally equal. -/
@@ -148,12 +171,15 @@ def hfdifferential {f : C^โโฎI, M; I', M'โฏ} {x : M} {y : M'} (h : f x = y)
map_smul' k v := rfl
map_add' v w := rfl
#align hfdifferential hfdifferential
+-/
+#print fdifferential /-
/-- The homogeneous differential as a linear map. -/
def fdifferential (f : C^โโฎI, M; I', M'โฏ) (x : M) :
PointDerivation I x โโ[๐] PointDerivation I' (f x) :=
hfdifferential (rfl : f x = f x)
#align fdifferential fdifferential
+-/
-- Standard notation for the differential. The abbreviation is `MId`.
scoped[Manifold] notation "๐
" => fdifferential
@@ -161,27 +187,33 @@ scoped[Manifold] notation "๐
" => fdifferential
-- Standard notation for the differential. The abbreviation is `MId`.
scoped[Manifold] notation "๐
โ" => hfdifferential
+#print apply_fdifferential /-
@[simp]
theorem apply_fdifferential (f : C^โโฎI, M; I', M'โฏ) {x : M} (v : PointDerivation I x)
(g : C^โโฎI', M'; ๐โฏ) : ๐
f x v g = v (g.comp f) :=
rfl
#align apply_fdifferential apply_fdifferential
+-/
+#print apply_hfdifferential /-
@[simp]
theorem apply_hfdifferential {f : C^โโฎI, M; I', M'โฏ} {x : M} {y : M'} (h : f x = y)
(v : PointDerivation I x) (g : C^โโฎI', M'; ๐โฏ) : ๐
โ h v g = ๐
f x v g :=
rfl
#align apply_hfdifferential apply_hfdifferential
+-/
variable {E'' : Type _} [NormedAddCommGroup E''] [NormedSpace ๐ E''] {H'' : Type _}
[TopologicalSpace H''] {I'' : ModelWithCorners ๐ E'' H''} {M'' : Type _} [TopologicalSpace M'']
[ChartedSpace H'' M'']
+#print fdifferential_comp /-
@[simp]
theorem fdifferential_comp (g : C^โโฎI', M'; I'', M''โฏ) (f : C^โโฎI, M; I', M'โฏ) (x : M) :
๐
(g.comp f) x = (๐
g (f x)).comp (๐
f x) :=
rfl
#align fdifferential_comp fdifferential_comp
+-/
end
mathlib commit https://github.com/leanprover-community/mathlib/commit/93f880918cb51905fd51b76add8273cbc27718ab
@@ -52,7 +52,7 @@ variable {๐ M}
namespace PointedSmoothMap
instance funLike {x : M} : FunLike C^โโฎI, M; ๐โฏโจxโฉ M fun _ => ๐ :=
- ContMdiffMap.funLike
+ ContMDiffMap.funLike
#align pointed_smooth_map.fun_like PointedSmoothMap.funLike
instance {x : M} : CommRing C^โโฎI, M; ๐โฏโจxโฉ :=
@@ -144,7 +144,7 @@ def hfdifferential {f : C^โโฎI, M; I', M'โฏ} {x : M} {y : M'} (h : f x = y)
simp only [SmoothMap.smul_comp, Derivation.map_smul, RingHom.id_apply] }
fun g g' => by
simp only [Derivation.leibniz, SmoothMap.mul_comp, LinearMap.coe_mk,
- PointedSmoothMap.smul_def, ContMdiffMap.comp_apply, h]
+ PointedSmoothMap.smul_def, ContMDiffMap.comp_apply, h]
map_smul' k v := rfl
map_add' v w := rfl
#align hfdifferential hfdifferential
mathlib commit https://github.com/leanprover-community/mathlib/commit/f2ad3645af9effcdb587637dc28a6074edc813f9
@@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Nicolรฒ Cavalleri
! This file was ported from Lean 3 source module geometry.manifold.derivation_bundle
-! leanprover-community/mathlib commit b608348ffaeb7f557f2fd46876037abafd326ff3
+! leanprover-community/mathlib commit 86c29aefdba50b3f33e86e52e3b2f51a0d8f0282
! Please do not edit these lines, except to modify the commit id
! if you have ported upstream changes.
-/
@@ -51,8 +51,9 @@ variable {๐ M}
namespace PointedSmoothMap
-instance {x : M} : CoeFun C^โโฎI, M; ๐โฏโจxโฉ fun _ => M โ ๐ :=
- ContMdiffMap.hasCoeToFun
+instance funLike {x : M} : FunLike C^โโฎI, M; ๐โฏโจxโฉ M fun _ => ๐ :=
+ ContMdiffMap.funLike
+#align pointed_smooth_map.fun_like PointedSmoothMap.funLike
instance {x : M} : CommRing C^โโฎI, M; ๐โฏโจxโฉ :=
SmoothMap.commRing
mathlib commit https://github.com/leanprover-community/mathlib/commit/9fb8964792b4237dac6200193a0d533f1b3f7423
@@ -45,7 +45,6 @@ def PointedSmoothMap (x : M) :=
C^nโฎI, M; ๐โฏ
#align pointed_smooth_map PointedSmoothMap
--- mathport name: pointed_smooth_map
scoped[Derivation] notation "C^" n "โฎ" I ", " M "; " ๐ "โฏโจ" x "โฉ" => PointedSmoothMap ๐ I M n x
variable {๐ M}
@@ -155,11 +154,9 @@ def fdifferential (f : C^โโฎI, M; I', M'โฏ) (x : M) :
hfdifferential (rfl : f x = f x)
#align fdifferential fdifferential
--- mathport name: fdifferential
-- Standard notation for the differential. The abbreviation is `MId`.
scoped[Manifold] notation "๐
" => fdifferential
--- mathport name: hfdifferential
-- Standard notation for the differential. The abbreviation is `MId`.
scoped[Manifold] notation "๐
โ" => hfdifferential
mathlib commit https://github.com/leanprover-community/mathlib/commit/34ebaffc1d1e8e783fc05438ec2e70af87275ac9
@@ -4,12 +4,12 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Nicolรฒ Cavalleri
! This file was ported from Lean 3 source module geometry.manifold.derivation_bundle
-! leanprover-community/mathlib commit a0735864ba72769da4b378673d3dbe2453924fde
+! leanprover-community/mathlib commit b608348ffaeb7f557f2fd46876037abafd326ff3
! Please do not edit these lines, except to modify the commit id
! if you have ported upstream changes.
-/
import Mathbin.Geometry.Manifold.Algebra.SmoothFunctions
-import Mathbin.RingTheory.Derivation
+import Mathbin.RingTheory.Derivation.Basic
/-!
mathlib commit https://github.com/leanprover-community/mathlib/commit/917c3c072e487b3cccdbfeff17e75b40e45f66cb
@@ -29,7 +29,7 @@ variable (๐ : Type _) [NontriviallyNormedField ๐] {E : Type _} [NormedAddC
[NormedSpace ๐ E] {H : Type _} [TopologicalSpace H] (I : ModelWithCorners ๐ E H) (M : Type _)
[TopologicalSpace M] [ChartedSpace H M] (n : โโ)
-open Manifold
+open scoped Manifold
-- the following two instances prevent poorly understood type class inference timeout problems
instance smoothFunctionsAlgebra : Algebra ๐ C^โโฎI, M; ๐โฏ := by infer_instance
@@ -92,7 +92,7 @@ instance (x : M) : IsScalarTower ๐ C^โโฎI, M; ๐โฏโจxโฉ ๐
end PointedSmoothMap
-open Derivation
+open scoped Derivation
/-- The derivations at a point of a manifold. Some regard this as a possible definition of the
tangent space -/
mathlib commit https://github.com/leanprover-community/mathlib/commit/bd9851ca476957ea4549eb19b40e7b5ade9428cc
@[inherit_doc]
on notations (#9942)
Make all the notations that unambiguously should inherit the docstring of their definition actually inherit it.
Also write a few docstrings by hand. I only wrote the ones I was competent to write and which I was sure of. Some docstrings come from mathlib3 as they were lost during the early port.
This PR is only intended as a first pass There are many more docstrings to add.
@@ -42,6 +42,7 @@ def PointedSmoothMap (_ : M) :=
C^nโฎI, M; ๐โฏ
#align pointed_smooth_map PointedSmoothMap
+@[inherit_doc]
scoped[Derivation] notation "C^" n "โฎ" I ", " M "; " ๐ "โฏโจ" x "โฉ" => PointedSmoothMap ๐ I M n x
variable {๐ M}
FunLike
(#9833)
This follows up from #9785, which renamed FunLike
to DFunLike
, by introducing a new abbreviation FunLike F ฮฑ ฮฒ := DFunLike F ฮฑ (fun _ => ฮฒ)
, to make the non-dependent use of FunLike
easier.
I searched for the pattern DFunLike.*fun
and DFunLike.*ฮป
in all files to replace expressions of the form DFunLike F ฮฑ (fun _ => ฮฒ)
with FunLike F ฮฑ ฮฒ
. I did this everywhere except for extends
clauses for two reasons: it would conflict with #8386, and more importantly extends
must directly refer to a structure with no unfolding of def
s or abbrev
s.
@@ -50,9 +50,9 @@ namespace PointedSmoothMap
open scoped Derivation
-instance instDFunLike {x : M} : DFunLike C^โโฎI, M; ๐โฏโจxโฉ M fun _ => ๐ :=
- ContMDiffMap.instDFunLike
-#align pointed_smooth_map.fun_like PointedSmoothMap.instDFunLike
+instance instFunLike {x : M} : FunLike C^โโฎI, M; ๐โฏโจxโฉ M ๐ :=
+ ContMDiffMap.instFunLike
+#align pointed_smooth_map.fun_like PointedSmoothMap.instFunLike
instance {x : M} : CommRing C^โโฎI, M; ๐โฏโจxโฉ :=
SmoothMap.commRing
FunLike
to DFunLike
(#9785)
This prepares for the introduction of a non-dependent synonym of FunLike, which helps a lot with keeping #8386 readable.
This is entirely search-and-replace in 680197f combined with manual fixes in 4145626, e900597 and b8428f8. The commands that generated this change:
sed -i 's/\bFunLike\b/DFunLike/g' {Archive,Counterexamples,Mathlib,test}/**/*.lean
sed -i 's/\btoFunLike\b/toDFunLike/g' {Archive,Counterexamples,Mathlib,test}/**/*.lean
sed -i 's/import Mathlib.Data.DFunLike/import Mathlib.Data.FunLike/g' {Archive,Counterexamples,Mathlib,test}/**/*.lean
sed -i 's/\bHom_FunLike\b/Hom_DFunLike/g' {Archive,Counterexamples,Mathlib,test}/**/*.lean
sed -i 's/\binstFunLike\b/instDFunLike/g' {Archive,Counterexamples,Mathlib,test}/**/*.lean
sed -i 's/\bfunLike\b/instDFunLike/g' {Archive,Counterexamples,Mathlib,test}/**/*.lean
sed -i 's/\btoo many metavariables to apply `fun_like.has_coe_to_fun`/too many metavariables to apply `DFunLike.hasCoeToFun`/g' {Archive,Counterexamples,Mathlib,test}/**/*.lean
Co-authored-by: Anne Baanen <Vierkantor@users.noreply.github.com>
@@ -50,9 +50,9 @@ namespace PointedSmoothMap
open scoped Derivation
-instance funLike {x : M} : FunLike C^โโฎI, M; ๐โฏโจxโฉ M fun _ => ๐ :=
- ContMDiffMap.funLike
-#align pointed_smooth_map.fun_like PointedSmoothMap.funLike
+instance instDFunLike {x : M} : DFunLike C^โโฎI, M; ๐โฏโจxโฉ M fun _ => ๐ :=
+ ContMDiffMap.instDFunLike
+#align pointed_smooth_map.fun_like PointedSmoothMap.instDFunLike
instance {x : M} : CommRing C^โโฎI, M; ๐โฏโจxโฉ :=
SmoothMap.commRing
Type _
and Sort _
(#6499)
We remove all possible occurences of Type _
and Sort _
in favor of Type*
and Sort*
.
This has nice performance benefits.
@@ -22,8 +22,8 @@ of the Lie algebra for a Lie group.
-/
-variable (๐ : Type _) [NontriviallyNormedField ๐] {E : Type _} [NormedAddCommGroup E]
- [NormedSpace ๐ E] {H : Type _} [TopologicalSpace H] (I : ModelWithCorners ๐ E H) (M : Type _)
+variable (๐ : Type*) [NontriviallyNormedField ๐] {E : Type*} [NormedAddCommGroup E]
+ [NormedSpace ๐ E] {H : Type*} [TopologicalSpace H] (I : ModelWithCorners ๐ E H) (M : Type*)
[TopologicalSpace M] [ChartedSpace H M] (n : โโ)
open scoped Manifold
@@ -127,8 +127,8 @@ theorem evalAt_apply (x : M) : evalAt x X f = (X f) x :=
end Derivation
-variable {I} {E' : Type _} [NormedAddCommGroup E'] [NormedSpace ๐ E'] {H' : Type _}
- [TopologicalSpace H'] {I' : ModelWithCorners ๐ E' H'} {M' : Type _} [TopologicalSpace M']
+variable {I} {E' : Type*} [NormedAddCommGroup E'] [NormedSpace ๐ E'] {H' : Type*}
+ [TopologicalSpace H'] {I' : ModelWithCorners ๐ E' H'} {M' : Type*} [TopologicalSpace M']
[ChartedSpace H' M']
/-- The heterogeneous differential as a linear map. Instead of taking a function as an argument this
@@ -176,8 +176,8 @@ theorem apply_hfdifferential {f : C^โโฎI, M; I', M'โฏ} {x : M} {y : M'} (h :
rfl
#align apply_hfdifferential apply_hfdifferential
-variable {E'' : Type _} [NormedAddCommGroup E''] [NormedSpace ๐ E''] {H'' : Type _}
- [TopologicalSpace H''] {I'' : ModelWithCorners ๐ E'' H''} {M'' : Type _} [TopologicalSpace M'']
+variable {E'' : Type*} [NormedAddCommGroup E''] [NormedSpace ๐ E''] {H'' : Type*}
+ [TopologicalSpace H''] {I'' : ModelWithCorners ๐ E'' H''} {M'' : Type*} [TopologicalSpace M'']
[ChartedSpace H'' M'']
@[simp]
@@ -2,15 +2,12 @@
Copyright ยฉ 2020 Nicolรฒ Cavalleri. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Nicolรฒ Cavalleri
-
-! This file was ported from Lean 3 source module geometry.manifold.derivation_bundle
-! leanprover-community/mathlib commit 86c29aefdba50b3f33e86e52e3b2f51a0d8f0282
-! Please do not edit these lines, except to modify the commit id
-! if you have ported upstream changes.
-/
import Mathlib.Geometry.Manifold.Algebra.SmoothFunctions
import Mathlib.RingTheory.Derivation.Basic
+#align_import geometry.manifold.derivation_bundle from "leanprover-community/mathlib"@"86c29aefdba50b3f33e86e52e3b2f51a0d8f0282"
+
/-!
# Derivation bundle
The unported dependencies are
algebra.order.module
init.core
linear_algebra.free_module.finite.rank
algebra.order.monoid.cancel.defs
algebra.abs
algebra.group_power.lemmas
init.data.list.basic
linear_algebra.free_module.rank
algebra.order.monoid.cancel.basic
init.data.list.default
topology.subset_properties
init.logic
The following 1 dependencies have changed in mathlib3 since they were ported, which may complicate porting this file