Skip to content

Commit

Permalink
feat(category_theory/sites): category of sheaves on the trivial topol…
Browse files Browse the repository at this point in the history
…ogy (#5651)

Shows that the category of sheaves on the trivial topology is just the category of presheaves.
  • Loading branch information
b-mehta committed Jan 7, 2021
1 parent 3c5d5c5 commit 18ba69b
Showing 1 changed file with 22 additions and 9 deletions.
31 changes: 22 additions & 9 deletions src/category_theory/sites/sheaf_of_types.lean
Expand Up @@ -687,6 +687,10 @@ begin
exact PK (pullback_arrows f R) (K.pullbacks f R hR) }
end

/-- Any presheaf is a sheaf for the bottom (trivial) grothendieck topology. -/
lemma is_sheaf_bot : is_sheaf (⊥ : grothendieck_topology C) P :=
λ X, by simp [is_sheaf_for_top_sieve]

end presieve

namespace equalizer
Expand Down Expand Up @@ -889,18 +893,27 @@ variables (J : grothendieck_topology C)
def SheafOfTypes (J : grothendieck_topology C) : Type (max u (v+1)) :=
{P : Cᵒᵖ ⥤ Type v // presieve.is_sheaf J P}

instance : inhabited (SheafOfTypes (⊥ : grothendieck_topology C)) :=
⟨⟨(functor.const _).obj punit,
λ X S hS,
begin
simp only [grothendieck_topology.bot_covering] at hS,
subst hS,
apply presieve.is_sheaf_for_top_sieve,
end⟩⟩

/-- The inclusion functor from sheaves to presheaves. -/
@[simps, derive [full, faithful]]
def SheafOfTypes_to_presheaf : SheafOfTypes J ⥤ (Cᵒᵖ ⥤ Type v) :=
full_subcategory_inclusion (presieve.is_sheaf J)

/--
The category of sheaves on the bottom (trivial) grothendieck topology is equivalent to the category
of presheaves.
-/
@[simps]
def SheafOfTypes_bot_equiv : SheafOfTypes (⊥ : grothendieck_topology C) ≌ (Cᵒᵖ ⥤ Type v) :=
{ functor := SheafOfTypes_to_presheaf _,
inverse :=
{ obj := λ P, ⟨P, presieve.is_sheaf_bot⟩,
map := λ P₁ P₂ f, (SheafOfTypes_to_presheaf _).preimage f },
unit_iso :=
{ hom := { app := λ _, 𝟙 _ },
inv := { app := λ _, 𝟙 _ } },
counit_iso := iso.refl _ }

instance : inhabited (SheafOfTypes (⊥ : grothendieck_topology C)) :=
⟨SheafOfTypes_bot_equiv.inverse.obj ((functor.const _).obj punit)⟩

end category_theory

0 comments on commit 18ba69b

Please sign in to comment.