Documentation

Mathlib.CategoryTheory.Sites.Coherent.LocallySurjective

Locally surjective morphisms of coherent sheaves #

This file characterises locally surjective morphisms of presheaves for the coherent, regular and extensive topologies.

Main results #

theorem CategoryTheory.regularTopology.isLocallySurjective_iff {C : Type u_1} (D : Type u_2) [CategoryTheory.Category.{u_3, u_1} C] [CategoryTheory.Category.{u_4, u_2} D] [CategoryTheory.ConcreteCategory D] [CategoryTheory.Preregular C] {F : CategoryTheory.Functor Cᵒᵖ D} {G : CategoryTheory.Functor Cᵒᵖ D} (f : F G) :
CategoryTheory.Presheaf.IsLocallySurjective (CategoryTheory.regularTopology C) f ∀ (X : C) (y : (CategoryTheory.forget D).obj (G.obj { unop := X })), ∃ (X' : C) (φ : X' X) (_ : CategoryTheory.EffectiveEpi φ) (x : (CategoryTheory.forget D).obj (F.obj { unop := X' })), (f.app { unop := X' }) x = (G.map { unop := φ }) y