Documentation

Mathlib.Algebra.Category.Grp.ForgetCorepresentable

The forget functor is corepresentable #

It is shown that the forget functor AddCommGrp.{u} ⥤ Type u is corepresentable by ULift. Similar results are obtained for the variants CommGrp, AddGrp and Grp.

(ULift ℤ →+ G) ≃ G #

These universe-monomorphic variants of zmultiplesHom/zpowersHom are put here since they shouldn't be useful outside of category theory.

The equivalence (ULift ℤ →+ G) ≃ G for any additive group G.

Equations
Instances For
    @[simp]
    theorem uliftZMultiplesHom_apply_apply (G : Type u) [AddGroup G] (a✝ : G) (a✝¹ : ULift.{u, 0} ) :
    ((uliftZMultiplesHom G) a✝) a✝¹ = AddEquiv.ulift a✝¹ a✝

    The equivalence (ULift (Multiplicative ℤ) →* G) ≃ G for any group G.

    Equations
    Instances For
      @[simp]
      theorem uliftZPowersHom_apply_apply (G : Type u) [Group G] (a✝ : G) (a✝¹ : ULift.{u, 0} (Multiplicative )) :
      ((uliftZPowersHom G) a✝) a✝¹ = a✝ ^ Multiplicative.toAdd (MulEquiv.ulift a✝¹)
      @[deprecated zpowersHom (since := "2025-05-11")]

      The equivalence (Multiplicative ℤ →* α) ≃ α for any group α.

      Equations
      Instances For
        @[deprecated uliftZPowersHom (since := "2025-05-11")]

        The equivalence (ULift (Multiplicative ℤ) →* α) ≃ α for any group α.

        Equations
        Instances For
          @[deprecated zmultiplesHom (since := "2025-05-11")]
          def AddMonoidHom.fromIntEquiv (α : Type u) [AddGroup α] :
          ( →+ α) α

          The equivalence (ℤ →+ α) ≃ α for any additive group α.

          Equations
          Instances For
            @[deprecated uliftZMultiplesHom (since := "2025-05-11")]

            The equivalence (ULift ℤ →+ α) ≃ α for any additive group α.

            Equations
            Instances For

              The forget functor Grp.{u} ⥤ Type u is corepresentable.

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

                The forget functor CommGrp.{u} ⥤ Type u is corepresentable.

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

                  The forget functor AddGrp.{u} ⥤ Type u is corepresentable.

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

                    The forget functor AddCommGrp.{u} ⥤ Type u is corepresentable.

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