The forget functor is corepresentable #
The forgetful functor AddCommMonCat.{u} ⥤ Type u
is corepresentable
by ULift ℕ
. Similar results are obtained for the variants CommMonCat
, AddMonCat
and MonCat
.
The equivalence (Multiplicative ℕ →* α) ≃ α
for any monoid α
.
Equations
- MonoidHom.fromMultiplicativeNatEquiv α = { toFun := fun (φ : Multiplicative ℕ →* α) => φ (Multiplicative.ofAdd 1), invFun := fun (x : α) => (powersHom α) x, left_inv := ⋯, right_inv := ⋯ }
Instances For
@[simp]
@[simp]
theorem
MonoidHom.fromMultiplicativeNatEquiv_apply
(α : Type u)
[Monoid α]
(φ : Multiplicative ℕ →* α)
:
The equivalence (ULift (Multiplicative ℕ) →* α) ≃ α
for any monoid α
.
Equations
Instances For
@[simp]
theorem
MonoidHom.fromULiftMultiplicativeNatEquiv_apply
(α : Type u)
[Monoid α]
(a✝ : ULift.{u, 0} (Multiplicative ℕ) →* α)
:
@[simp]
theorem
MonoidHom.fromULiftMultiplicativeNatEquiv_symm_apply_apply
(α : Type u)
[Monoid α]
(a✝ : α)
(a✝¹ : ULift.{u, 0} (Multiplicative ℕ))
:
The equivalence (ℤ →+ α) ≃ α
for any additive group α
.
Equations
- AddMonoidHom.fromNatEquiv α = { toFun := fun (φ : ℕ →+ α) => φ 1, invFun := fun (x : α) => (multiplesHom α) x, left_inv := ⋯, right_inv := ⋯ }
Instances For
@[simp]
@[simp]
The equivalence (ULift ℕ →+ α) ≃ α
for any additive monoid α
.
Equations
Instances For
@[simp]
theorem
AddMonoidHom.fromULiftNatEquiv_apply
(α : Type u)
[AddMonoid α]
(a✝ : ULift.{u, 0} ℕ →+ α)
:
@[simp]
theorem
AddMonoidHom.fromULiftNatEquiv_symm_apply_apply
(α : Type u)
[AddMonoid α]
(a✝ : α)
(a✝¹ : ULift.{u, 0} ℕ)
:
The forgetful functor MonCat.{u} ⥤ Type u
is corepresentable.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The forgetful functor CommMonCat.{u} ⥤ Type u
is corepresentable.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The forgetful functor AddMonCat.{u} ⥤ Type u
is corepresentable.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The forgetful functor AddCommMonCat.{u} ⥤ Type u
is corepresentable.
Equations
- One or more equations did not get rendered due to their size.