Here we construct the natural model for groupoids.
TODO: This file needs to eventually be ported to GroupoidRussellNaturalModel but currently we don't have a Russell style sigma type.
Equations
Instances For
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
Instances For
Equations
Instances For
Equations
Instances For
def
PshsGrpdOfPshGrpd :
CategoryTheory.Functor (CategoryTheory.Functor CategoryTheory.Grpdᵒᵖ (Type (u + 1)))
(CategoryTheory.Functor sGrpdᵒᵖ (Type (u + 1)))
Equations
Instances For
@[reducible, inline]
Equations
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
theorem
yonedaCatEquiv_naturality
{Γ Δ : sGrpd}
{C : Type (u + 1)}
[CategoryTheory.Category.{u, u + 1} C]
(A : CategoryTheory.yoneda.obj Γ ⟶ yonedaCat.obj (CategoryTheory.Cat.of C))
(σ : Δ ⟶ Γ)
:
@[reducible, inline]
Equations
Instances For
@[reducible, inline]
Equations
Instances For
@[reducible, inline]
Instances For
Equations
- One or more equations did not get rendered due to their size.
Equations
- groupoidULift = CategoryTheory.Groupoid.mk (fun {X Y : ULift.{?u.22, ?u.24} α} (f : X ⟶ Y) => CategoryTheory.Groupoid.inv f) ⋯ ⋯
Equations
- groupoidULiftHom = CategoryTheory.Groupoid.mk (fun {X Y : CategoryTheory.ULiftHom α} (f : X ⟶ Y) => { down := CategoryTheory.Groupoid.inv f.down }) ⋯ ⋯
A model of Grpd with an internal universe, with the property that the small universe injects into the large one.
Instances For
def
PointToFiber
{Γ : CategoryTheory.Grpd}
(A : CategoryTheory.Functor (↑Γ) CategoryTheory.Grpd)
(x : ↑Γ)
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
PointToFiberNT
{Γ : CategoryTheory.Grpd}
(A : CategoryTheory.Functor (↑Γ) CategoryTheory.Grpd)
(X Y : ↑Γ)
(f : X ⟶ Y)
:
Equations
- PointToFiberNT A X Y f = { app := fun (x : ↑(A.obj X)) => { base := id f, fiber := id (CategoryTheory.CategoryStruct.id ((A.map f).obj x)) }, naturality := ⋯ }
Instances For
Instances For
def
GroupoidSigma
(Γ : CategoryTheory.Grpd)
(A : CategoryTheory.Functor (↑Γ) CategoryTheory.Grpd)
(B : CategoryTheory.Functor (CategoryTheory.Grothendieck.Groupoidal A) CategoryTheory.Grpd)
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
GroupoidSigmaMake
{Γ : CategoryTheory.Grpd}
{A : CategoryTheory.Functor (↑Γ) CategoryTheory.Grpd}
{B : CategoryTheory.Functor (CategoryTheory.Grothendieck.Groupoidal A) CategoryTheory.Grpd}
{x : ↑Γ}
(Ax : ↑(A.obj x))
(Bx : ↑(B.obj { base := x, fiber := Ax }))
:
↑((GroupoidSigma Γ A B).obj x)
Equations
- GroupoidSigmaMake Ax Bx = { base := Ax, fiber := Bx }
Instances For
def
GroupoidSigmaBase
(Γ : CategoryTheory.Grpd)
(A : CategoryTheory.Functor (↑Γ) CategoryTheory.Grpd)
(B : CategoryTheory.Functor (CategoryTheory.Grothendieck.Groupoidal A) CategoryTheory.Grpd)
:
Equations
- GroupoidSigmaBase Γ A B = { app := id fun (x : ↑Γ) => id sorry, naturality := ⋯ }
Instances For
theorem
GroupoidSigmaBeckChevalley
(Δ Γ : CategoryTheory.Grpd)
(σ : CategoryTheory.Functor ↑Δ ↑Γ)
(A : CategoryTheory.Functor (↑Γ) CategoryTheory.Grpd)
(B : CategoryTheory.Functor (CategoryTheory.Grothendieck.Groupoidal A) CategoryTheory.Grpd)
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
Instances For
instance
instGroupoidFunctor_groupoidModel
(G1 G2 : Type)
[CategoryTheory.Groupoid G1]
[CategoryTheory.Groupoid G2]
:
Equations
- One or more equations did not get rendered due to their size.
def
GroupoidPiMap
(Γ : CategoryTheory.Grpd)
(A : CategoryTheory.Functor (↑Γ) CategoryTheory.Grpd)
(B : CategoryTheory.Functor (CategoryTheory.Grothendieck.Groupoidal A) CategoryTheory.Grpd)
:
Equations
- One or more equations did not get rendered due to their size.
Instances For
def
GroupoidPi
(Γ : CategoryTheory.Grpd)
(A : CategoryTheory.Functor (↑Γ) CategoryTheory.Grpd)
(B : CategoryTheory.Functor (CategoryTheory.Grothendieck.Groupoidal A) CategoryTheory.Grpd)
:
Equations
- One or more equations did not get rendered due to their size.