Skip to content

Commit

Permalink
feat: big Zariski is subcanonical (#12028)
Browse files Browse the repository at this point in the history
  • Loading branch information
adamtopaz committed Apr 9, 2024
1 parent aee79f6 commit e8433a6
Showing 1 changed file with 21 additions and 1 deletion.
22 changes: 21 additions & 1 deletion Mathlib/AlgebraicGeometry/Sites/BigZariski.lean
Original file line number Diff line number Diff line change
@@ -1,10 +1,11 @@
/-
Copyright (c) 2023 Joël Riou. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Joël Riou
Authors: Joël Riou, Adam Topaz
-/
import Mathlib.AlgebraicGeometry.Pullbacks
import Mathlib.CategoryTheory.Sites.Pretopology
import Mathlib.CategoryTheory.Sites.Canonical
/-!
# The big Zariski site of schemes
Expand Down Expand Up @@ -69,6 +70,25 @@ lemma zariskiTopology_openCover {Y : Scheme.{u}} (U : OpenCover.{v} Y) :
rintro _ _ ⟨y⟩
exact ⟨_, 𝟙 _, U.map (U.f y), ⟨_⟩, by simp⟩

lemma subcanonical_zariskiTopology : Sheaf.Subcanonical zariskiTopology := by
apply Sheaf.Subcanonical.of_yoneda_isSheaf
intro X
rw [Presieve.isSheaf_pretopology]
rintro Y S ⟨𝓤,rfl⟩ x hx
let e : Y ⟶ X := 𝓤.glueMorphisms (fun j => x (𝓤.map _) (.mk _)) <| by
intro i j
apply hx
exact Limits.pullback.condition
refine ⟨e, ?_, ?_⟩
· rintro Z e ⟨j⟩
dsimp [e]
rw [𝓤.ι_glueMorphisms]
· intro e' h
apply 𝓤.hom_ext
intro j
rw [𝓤.ι_glueMorphisms]
exact h (𝓤.map j) (.mk j)

end Scheme

end AlgebraicGeometry

0 comments on commit e8433a6

Please sign in to comment.