Continuous functors between sites. #
We define the notion of continuous functor between sites: these are functors F such that
the precomposition with F.op preserves sheaves of types (and actually sheaves in any
category).
Main definitions #
Functor.IsContinuous: a functor between sites is continuous if the precomposition with this functor preserves sheaves with values in the categoryType tfor a certain auxiliary universet.Functor.sheafPushforwardContinuous: the induced functorSheaf K A ⥤ Sheaf J Afor a continuous functorG : (C, J) ⥤ (D, K). In case this is part of a morphism of sites, this would be understood as the pushforward functor even though it goes in the opposite direction as the functorG. (Here, the auxiliary universetin the assumption thatGis continuous is the one such that morphisms in the categoryAare inType t.)Functor.PreservesOneHypercovers: a type-class expressing that a functor preserves 1-hypercovers of a certain size
Main result #
Functor.isContinuous_of_preservesOneHypercovers: if the topology onCis generated by 1-hypercovers of sizewand thatF : C ⥤ Dpreserves 1-hypercovers of sizew, thenFis continuous (for any auxiliary universe parametert). This is an instance forw = max u₁ v₁whenC : Type u₁and[Category.{v₁} C]
References #
The image of a 1-pre-hypercover by a functor.
Equations
- One or more equations did not get rendered due to their size.
Instances For
If F : C ⥤ D, P : Dᵒᵖ ⥤ A and E is a 1-pre-hypercover of an object of X,
then (E.map F).multifork P is a limit iff E.multifork (F.op ⋙ P) is a limit.
Equations
- E.isLimitMapMultiforkEquiv F P = Equiv.refl (CategoryTheory.Limits.IsLimit ((E.map F).multifork P))
Instances For
A 1-hypercover in C is preserved by a functor F : C ⥤ D if the mapped 1-pre-hypercover
in D is a 1-hypercover for the given topology on D.
Instances
Given a 1-hypercover E : J.OneHypercover X of an object of C, a functor F : C ⥤ D
such that E.IsPreservedBy F K for a Grothendieck topology K on D, this is
the image of E by F, as a 1-hypercover of F.obj X for K.
Instances For
The condition that a functor F : C ⥤ D sends 1-hypercovers for
J : GrothendieckTopology C to 1-hypercovers for K : GrothendieckTopology D.
Equations
- F.PreservesOneHypercovers J K = ∀ {X : C} (E : J.OneHypercover X), E.IsPreservedBy F K
Instances For
A functor F is continuous if the precomposition with F.op sends sheaves of Type t
to sheaves.
Instances
The induced functor Sheaf K A ⥤ Sheaf J A given by F.op ⋙ _
if F is a continuous functor.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The functor F.sheafPushforwardContinuous A J K : Sheaf K A ⥤ Sheaf J A
is induced by the precomposition with F.op.
Equations
Instances For
The functor sheafPushforwardContinuous corresponding to the identity functor
identifies to the identity functor.
Equations
Instances For
The composition of two pushforward functors on sheaves identifies to the pushforward for the composition of the two functors.
Equations
- F.sheafPushforwardContinuousComp G A J K L = CategoryTheory.Iso.refl ((G.sheafPushforwardContinuous A K L).comp (F.sheafPushforwardContinuous A J K))
Instances For
The action of a natural transformation on pushforward functors of sheaves.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The action of a natural isomorphism on pushforward functors of sheaves.
Equations
- One or more equations did not get rendered due to their size.
Instances For
If a continuous functor between sites is isomorphic to the identity functor, then the corresponding pushforward functor on sheaves identifies to the identity functor.
Equations
Instances For
When we have an isomorphism F ⋙ G ≅ FG between continuous functors
between sites, the composition of the pushforward functors for
G and F identifies to the pushforward functor for FG.
Equations
- CategoryTheory.Functor.sheafPushforwardContinuousComp' eFG A J K L = F.sheafPushforwardContinuousComp G A J K L ≪≫ CategoryTheory.Functor.sheafPushforwardContinuousIso eFG A J L