module Cat.Displayed.Bifibration
{o ℓ o' ℓ'} {ℬ : Precategory o ℓ} (ℰ : Displayed ℬ o' ℓ') where
Bifibrations🔗
A displayed category is a bifibration if is it both a fibration and an opfibration. This means that is equipped with both reindexing and opreindexing functors, which allows us to both restrict and extend along morphisms in the base.
Note that a bifibration is not the same as a “profunctor valued in categories”. Those are a distinct concept, called two-sided fibrations.
record is-bifibration : Type (o ⊔ ℓ ⊔ o' ⊔ ℓ') where
field
: Cartesian-fibration
fibration : Cocartesian-fibration
opfibration
module fibration = Cartesian-fibration fibration
module opfibration = Cocartesian-fibration opfibration
Bifibrations and adjoints🔗
If is a bifibration, then its opreindexing functors are left adjoints to its reindexing functors. To show this, it will suffice to construct natural isomorphism between and However, we have already shown that and are both naturally isomorphic to 1, so all we need to do is compose these natural isomorphisms!
module _ (bifib : is-bifibration) where
open is-bifibration bifib
open Cat.Displayed.Cartesian.Indexing ℰ fibration
open Cat.Displayed.Cocartesian.Indexing ℰ opfibration
cobase-change⊣base-change: ∀ {x y} (f : Hom x y)
→ cobase-change f ⊣ base-change f
{x} {y} f =
cobase-change⊣base-change
hom-natural-iso→adjoints $(opfibration→hom-iso opfibration f ni⁻¹) ∘ni fibration→hom-iso fibration f
In fact, if is a cartesian fibration where every reindexing functor has a left adjoint, then is a bifibration!
Since is a fibration, every in induces a natural isomorphism by the universal property of cartesian lifts. If additionally has a left adjoint we have natural isomorphisms
which implies
is a weak opfibration
; and any
weak opfibration that’s also a fibration is a proper opfibration.
module _ (fib : Cartesian-fibration) where
open Cartesian-fibration fib
open Cat.Displayed.Cartesian.Indexing ℰ fib
left-adjoint-base-change→opfibration: (L : ∀ {x y} → (f : Hom x y) → Functor (Fibre ℰ x) (Fibre ℰ y))
→ (∀ {x y} → (f : Hom x y) → (L f ⊣ base-change f))
→ Cocartesian-fibration
=
left-adjoint-base-change→opfibration L adj
cartesian+weak-opfibration→opfibration fib $λ u →
hom-iso→weak-opfibration L (adjunct-hom-iso-from (adj u) _ ni⁻¹) fibration→hom-iso-from fib u ∘ni
Adjoints from cocartesian maps🔗
Let be a morphism in and let be a functor. If we are given a natural transformation with cocartesian, then is a left adjoint to
cocartesian→left-adjoint-base-change: ∀ {x y} {L : Functor (Fibre ℰ x) (Fibre ℰ y)} {f : Hom x y}
→ (L-unit : Id => base-change f F∘ L)
→ (∀ x → is-cocartesian (f ∘ id) (has-lift.lifting f (L .F₀ x) ∘' L-unit .η x))
→ L ⊣ base-change f
We will construct the adjunction by constructing a natural equivalence of
The map gives us the forward direction of this equivalence, so all that remains is to find an inverse. Since is cocartesian, it satisfies a mapping-out universal property: if is a vertical map in we can construct a vertical map by factoring through the cocartesian The actual universal property says that this factorising process is an equivalence.
{x = x} {y = y} {L = L} {f = f} L-unit cocart =
cocartesian→left-adjoint-base-change (λ v → base-change f .F₁ v Fib.∘ L-unit .η _)
hom-iso→adjoints where
precompose-equiv equiv-natural module cocart x = is-cocartesian (cocart x)
module f* = Functor (base-change f)
precompose-equiv: ∀ {x' : Ob[ x ]} {y' : Ob[ y ]}
→ is-equiv {A = Hom[ id ] (L .F₀ x') y'} (λ v → f*.₁ v Fib.∘ L-unit .η x')
{x'} {y'} = is-iso→is-equiv $ iso
precompose-equiv (λ v → cocart.universalv _ (has-lift.lifting f _ ∘' v))
(λ v → has-lift.uniquep₂ _ _ _ _ refl _ _
(Fib.pulllf (has-lift.commutesp f _ id-comm _)
(assoc' _ _ _)
∙[] symP .commutesv x' _)
∙[] cocart)
refl(λ v → symP $ cocart.uniquep x' _ _ _ _ $
_ _ _
assoc' .pushlf (symP $ has-lift.commutesp f _ id-comm _)) ∙[] Fib
Futhermore, this equivalence is natural, but that’s a very tedious proof.
equiv-natural: hom-iso-natural {L = L} {R = base-change f} (λ v → f*.₁ v Fib.∘ L-unit .η _)
=
equiv-natural g h k .uniquep₂ _ _ _ _ _ _ _
has-lift(Fib.pulllf (has-lift.commutesp f _ id-comm _)
_ (pushl[] _ (to-pathp⁻ (smashr _ _))))
∙[] pushl[] (Fib.pulllf (has-lift.commutesp f _ id-comm _)
_ (Fib.pulllf (Fib.pulllf (has-lift.commutesp f _ id-comm _)))
∙[] extendr[] _ (pullr[] _ (to-pathp (L-unit .is-natural _ _ h)))
∙[] extendr[] _ (Fib.pulllf (extendr[] _ (has-lift.commutesp f _ id-comm _)))) ∙[] pullr[]
see
opfibration→hom-iso
andfibration→hom-iso
.↩︎