Documentation

Mathlib.Algebra.Category.ModuleCat.Adjunctions

The functor of forming finitely supported functions on a type with values in a [Ring R] is the left adjoint of the forgetful functor from R-modules to types.

@[simp]
theorem ModuleCat.free_map (R : Type u) [Ring R] {X : Type u} {Y : Type u} (f : X Y) :
@[simp]
theorem ModuleCat.free_obj (R : Type u) [Ring R] (X : Type u) :

The free functor Type u ⥤ ModuleCat R sending a type X to the free R-module with generators x : X, implemented as the type X →₀ R.

Equations
Instances For

    The free-forgetful adjunction for R-modules.

    Equations
    • One or more equations did not get rendered due to their size.
    Instances For
      Equations
      • =
      def ModuleCat.Free.ε (R : Type u) [CommRing R] :
      𝟙_ (ModuleCat R) (ModuleCat.free R).obj (𝟙_ (Type u))

      (Implementation detail) The unitor for Free R.

      Equations
      Instances For

        (Implementation detail) The tensorator for Free R.

        Equations
        Instances For
          @[simp]
          theorem ModuleCat.Free.instLaxMonoidalObjFree_ε (R : Type u) [CommRing R] :
          CategoryTheory.LaxMonoidal.ε = ModuleCat.Free.ε R

          The free R-module functor is lax monoidal.

          Equations
          instance ModuleCat.Free.instIsIsoε (R : Type u) [CommRing R] :
          CategoryTheory.IsIso CategoryTheory.LaxMonoidal.ε
          Equations
          • =

          The free functor Type u ⥤ ModuleCat R, as a monoidal functor.

          Equations
          Instances For
            def CategoryTheory.Free :
            Type u_1 → Type u → Type u

            Free R C is a type synonym for C, which, given [CommRing R] and [Category C], we will equip with a category structure where the morphisms are formal R-linear combinations of the morphisms in C.

            Equations
            Instances For
              def CategoryTheory.Free.of (R : Type u_1) {C : Type u} (X : C) :

              Consider an object of C as an object of the R-linear completion.

              It may be preferable to use (Free.embedding R C).obj X instead; this functor can also be used to lift morphisms.

              Equations
              Instances For
                Equations
                Equations
                @[simp]
                theorem CategoryTheory.Free.embedding_map (R : Type u_1) [CommRing R] (C : Type u) [CategoryTheory.Category.{v, u} C] {X : C} {Y : C} (f : X Y) :

                A category embeds into its R-linear completion.

                Equations
                Instances For

                  A functor to an R-linear category lifts to a functor from its R-linear completion.

                  Equations
                  • One or more equations did not get rendered due to their size.
                  Instances For

                    The embedding into the R-linear completion, followed by the lift, is isomorphic to the original functor.

                    Equations
                    • One or more equations did not get rendered due to their size.
                    Instances For

                      Two R-linear functors out of the R-linear completion are isomorphic iff their compositions with the embedding functor are isomorphic.

                      Equations
                      Instances For

                        Free.lift is unique amongst R-linear functors Free R C ⥤ D which compose with embedding ℤ C to give the original functor.

                        Equations
                        Instances For