Documentation

Mathlib.CategoryTheory.Sites.Coherent.RegularSheaves

Sheaves for the regular topology #

This file characterises sheaves for the regular topology.

Main results #

A presieve is regular if it consists of a single effective epimorphism.

Instances

    A contravariant functor on C satisifies SingleEqualizerCondition with respect to a morphism π if it takes its kernel pair to an equalizer diagram.

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

      A contravariant functor on C satisfies EqualizerCondition if it takes kernel pairs of effective epimorphisms to equalizer diagrams.

      Equations
      Instances For
        def CategoryTheory.regularTopology.MapToEqualizer {C : Type u_1} [CategoryTheory.Category.{u_5, u_1} C] (P : CategoryTheory.Functor Cᵒᵖ (Type u_4)) {W : C} {X : C} {B : C} (f : X B) (g₁ : W X) (g₂ : W X) (w : CategoryTheory.CategoryStruct.comp g₁ f = CategoryTheory.CategoryStruct.comp g₂ f) :
        P.obj (Opposite.op B){x : P.obj (Opposite.op X) | P.map g₁.op x = P.map g₂.op x}

        The canonical map to the explicit equalizer.

        Equations
        Instances For
          theorem CategoryTheory.regularTopology.equalizerCondition_w' {C : Type u_1} [CategoryTheory.Category.{u_5, u_1} C] (P : CategoryTheory.Functor Cᵒᵖ (Type u_4)) {X : C} {B : C} (π : X B) [CategoryTheory.Limits.HasPullback π π] :
          CategoryTheory.CategoryStruct.comp (P.map π.op) (P.map CategoryTheory.Limits.pullback.fst.op) = CategoryTheory.CategoryStruct.comp (P.map π.op) (P.map CategoryTheory.Limits.pullback.snd.op)
          theorem CategoryTheory.regularTopology.mapToEqualizer_eq_comp {C : Type u_1} [CategoryTheory.Category.{u_5, u_1} C] (P : CategoryTheory.Functor Cᵒᵖ (Type u_4)) {X : C} {B : C} (π : X B) [CategoryTheory.Limits.HasPullback π π] :
          CategoryTheory.regularTopology.MapToEqualizer P π CategoryTheory.Limits.pullback.fst CategoryTheory.Limits.pullback.snd = CategoryTheory.CategoryStruct.comp (CategoryTheory.Limits.equalizer.lift (P.map π.op) ) (CategoryTheory.Limits.Types.equalizerIso (P.map CategoryTheory.Limits.pullback.fst.op) (P.map CategoryTheory.Limits.pullback.snd.op)).hom

          An alternative phrasing of the explicit equalizer condition, using more categorical language.

          Given a limiting pullback cone, the fork in SingleEqualizerCondition is limiting iff the diagram in Presheaf.isSheaf_iff_isLimit_coverage is limiting.

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

            Every Yoneda-presheaf is a sheaf for the regular topology.