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.
The content of this file is not meant to be regarded as an alternative definition to the current tangent bundle but rather as a purely algebraic theory that provides a purely algebraic definition of the Lie algebra for a Lie group.
Equations
Type synonym, introduced to put a different has_smul
action on C^n⟮I, M; 𝕜⟯
which is defined as f • r = f(x) * r
.
Equations
- pointed_smooth_map 𝕜 I M n x = cont_mdiff_map I (model_with_corners_self 𝕜 𝕜) M 𝕜 n
Instances for pointed_smooth_map
Equations
Equations
Equations
Equations
- pointed_smooth_map.inhabited I = {default := 0}
Equations
smooth_map.eval_ring_hom
gives rise to an algebra structure of C^∞⟮I, M; 𝕜⟯
on 𝕜
.
Equations
With the eval_algebra
algebra structure evaluation is actually an algebra morphism.
Equations
- pointed_smooth_map.eval x = algebra.of_id (pointed_smooth_map 𝕜 I M ⊤ x) 𝕜
The derivations at a point of a manifold. Some regard this as a possible definition of the tangent space
Equations
- point_derivation I x = derivation 𝕜 (pointed_smooth_map 𝕜 I M ⊤ x) 𝕜
Evaluation at a point gives rise to a C^∞⟮I, M; 𝕜⟯
-linear map between C^∞⟮I, M; 𝕜⟯
and 𝕜
.
Equations
The evaluation at a point as a linear map.
Equations
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.
Equations
- hfdifferential h = {to_fun := λ (v : point_derivation I x), derivation.mk' {to_fun := λ (g : pointed_smooth_map 𝕜 I' M' ⊤ y), ⇑v (cont_mdiff_map.comp g f), map_add' := _, map_smul' := _} _, map_add' := _, map_smul' := _}
The homogeneous differential as a linear map.
Equations
- fdifferential f x = hfdifferential _