Skip to content

Commit

Permalink
refactor(algebraic_geometry/*): rename structure sheaf to `Spec.struc…
Browse files Browse the repository at this point in the history
…ture_sheaf` (#12785)

Following [this Zulip message](https://leanprover.zulipchat.com/#narrow/stream/113488-general/topic/Rename.20.60structure_sheaf.60.20to.20.60Spec.2Estructure_sheaf.60/near/275649595), this pr renames `structure_sheaf` to `Spec.structure_sheaf`
  • Loading branch information
jjaassoonn committed Mar 23, 2022
1 parent 16fb8e2 commit 84a438e
Show file tree
Hide file tree
Showing 4 changed files with 6 additions and 3 deletions.
2 changes: 2 additions & 0 deletions src/algebraic_geometry/AffineScheme.lean
Expand Up @@ -37,6 +37,8 @@ universe u

namespace algebraic_geometry

open Spec (structure_sheaf)

/-- The category of affine schemes -/
def AffineScheme := Scheme.Spec.ess_image

Expand Down
2 changes: 1 addition & 1 deletion src/algebraic_geometry/Gamma_Spec_adjunction.lean
Expand Up @@ -38,7 +38,7 @@ open prime_spectrum
namespace algebraic_geometry
open opposite
open category_theory
open structure_sheaf
open structure_sheaf Spec (structure_sheaf)
open topological_space
open algebraic_geometry.LocallyRingedSpace
open Top.presheaf
Expand Down
2 changes: 1 addition & 1 deletion src/algebraic_geometry/Spec.lean
Expand Up @@ -38,7 +38,7 @@ universes u v
namespace algebraic_geometry
open opposite
open category_theory
open structure_sheaf
open structure_sheaf Spec (structure_sheaf)

/--
The spectrum of a commutative ring, as a topological space.
Expand Down
3 changes: 2 additions & 1 deletion src/algebraic_geometry/structure_sheaf.lean
Expand Up @@ -257,13 +257,14 @@ The structure sheaf on $Spec R$, valued in `CommRing`.
This is provided as a bundled `SheafedSpace` as `Spec.SheafedSpace R` later.
-/
def structure_sheaf : sheaf CommRing (prime_spectrum.Top R) :=
def Spec.structure_sheaf : sheaf CommRing (prime_spectrum.Top R) :=
⟨structure_presheaf_in_CommRing R,
-- We check the sheaf condition under `forget CommRing`.
(is_sheaf_iff_is_sheaf_comp _ _).mpr
(is_sheaf_of_iso (structure_presheaf_comp_forget R).symm
(structure_sheaf_in_Type R).property)⟩

open Spec (structure_sheaf)

namespace structure_sheaf

Expand Down

0 comments on commit 84a438e

Please sign in to comment.