Documentation

Mathlib.Geometry.Manifold.Algebra.Structures

Smooth structures #

In this file we define smooth structures that build on Lie groups. We prefer using the term smooth instead of Lie mainly because Lie ring has currently another use in mathematics.

class SmoothRing {𝕜 : Type u_1} [NontriviallyNormedField 𝕜] {H : Type u_2} [TopologicalSpace H] {E : Type u_3} [NormedAddCommGroup E] [NormedSpace 𝕜 E] (I : ModelWithCorners 𝕜 E H) (R : Type u_4) [Semiring R] [TopologicalSpace R] [ChartedSpace H R] extends SmoothAdd :

A smooth (semi)ring is a (semi)ring R where addition and multiplication are smooth. If R is a ring, then negation is automatically smooth, as it is multiplication with -1.

Instances
    instance SmoothRing.toSmoothMul {𝕜 : Type u_1} [NontriviallyNormedField 𝕜] {H : Type u_2} [TopologicalSpace H] {E : Type u_3} [NormedAddCommGroup E] [NormedSpace 𝕜 E] (I : ModelWithCorners 𝕜 E H) (R : Type u_4) [Semiring R] [TopologicalSpace R] [ChartedSpace H R] [h : SmoothRing I R] :
    Equations
    • =
    instance SmoothRing.toLieAddGroup {𝕜 : Type u_1} [NontriviallyNormedField 𝕜] {H : Type u_2} [TopologicalSpace H] {E : Type u_3} [NormedAddCommGroup E] [NormedSpace 𝕜 E] (I : ModelWithCorners 𝕜 E H) (R : Type u_4) [Ring R] [TopologicalSpace R] [ChartedSpace H R] [SmoothRing I R] :
    Equations
    • =
    instance fieldSmoothRing {𝕜 : Type u_1} [NontriviallyNormedField 𝕜] :
    Equations
    • =

    A smooth (semi)ring is a topological (semi)ring. This is not an instance for technical reasons, see note [Design choices about smooth algebraic structures].