Skip to content
This repository has been archived by the owner on Jul 24, 2024. It is now read-only.

[Merged by Bors] - feature(algebraic_geometry/Scheme): the category of schemes #3961

Closed
wants to merge 181 commits into from

Conversation

semorrison
Copy link
Collaborator

@semorrison semorrison commented Aug 28, 2020

The definition of a Scheme, and the category of schemes as the full subcategory of locally ringed spaces.

Co-authored-by: Johan Commelin johan@commelin.net


Blocked #3609, #3906, #3907

kbuzzard and others added 30 commits July 23, 2020 23:10
Co-authored-by: Markus Himmel <markus@himmel-villmar.de>
@github-actions github-actions bot removed the merge-conflict Please `git merge origin/master` then a bot will remove this label. label Aug 30, 2020
@semorrison semorrison added the awaiting-review The author would like community review of the PR label Aug 30, 2020
src/algebra/ring/basic.lean Show resolved Hide resolved
src/topology/opens.lean Outdated Show resolved Hide resolved

@[ext] lemma ext {X Y : PresheafedSpace C} (α β : hom X Y)
(w : α.base = β.base) (h : α.c ≫ (whisker_right (nat_trans.op (opens.map_iso _ _ w).inv) X.𝒪) = β.c) :
(w : α.base = β.base)
(h : α.c ≫ (whisker_right (nat_trans.op (opens.map_iso _ _ w).inv) X.presheaf) = β.c) :
Copy link
Collaborator

Choose a reason for hiding this comment

The reason will be displayed to describe this comment to others. Learn more.

Is this the solution to the problem of equality of types?

Copy link
Collaborator Author

Choose a reason for hiding this comment

The reason will be displayed to describe this comment to others. Learn more.

I'm sorry, could you clarify your question, I'm not sure how it relates to this piece of the code.

Copy link
Collaborator

Choose a reason for hiding this comment

The reason will be displayed to describe this comment to others. Learn more.

Well, equality of types proved to be troublesome, but somehow you managed to use it without issues. (α.base = β.base is an equality of types right)

Comment on lines 47 to 48
/-- The structure sheaf of a locally ringed space. -/
def 𝒪 : sheaf CommRing X.to_Top := ⟨X.1.presheaf, X.1.sheaf_condition⟩
Copy link
Collaborator

Choose a reason for hiding this comment

The reason will be displayed to describe this comment to others. Learn more.

Why not coerce X to a sheafed space?

Copy link
Collaborator Author

Choose a reason for hiding this comment

The reason will be displayed to describe this comment to others. Learn more.

I can't do exactly that, but I've replaced the RHS with X.to_SheafedSpace.sheaf. Is that okay?

Copy link
Collaborator

Choose a reason for hiding this comment

The reason will be displayed to describe this comment to others. Learn more.

Sure, but why do we not prefer coercion?

src/ring_theory/ideal/basic.lean Outdated Show resolved Hide resolved
src/algebraic_geometry/prime_spectrum.lean Outdated Show resolved Hide resolved
src/algebraic_geometry/prime_spectrum.lean Outdated Show resolved Hide resolved
src/algebraic_geometry/structure_sheaf.lean Outdated Show resolved Hide resolved
src/algebraic_geometry/structure_sheaf.lean Show resolved Hide resolved
src/algebraic_geometry/structure_sheaf.lean Outdated Show resolved Hide resolved
src/algebraic_geometry/presheafed_space.lean Outdated Show resolved Hide resolved
src/algebraic_geometry/stalks.lean Outdated Show resolved Hide resolved
src/algebraic_geometry/prime_spectrum.lean Show resolved Hide resolved
src/algebraic_geometry/presheafed_space.lean Outdated Show resolved Hide resolved
src/algebraic_geometry/presheafed_space.lean Outdated Show resolved Hide resolved
src/algebraic_geometry/presheafed_space.lean Outdated Show resolved Hide resolved
Co-authored-by: Bryan Gin-ge Chen <bryangingechen@gmail.com>
@PatrickMassot
Copy link
Member

bors merge

@github-actions github-actions bot added ready-to-merge All that is left is for bors to build and merge this PR. (Remember you need to say `bors r+`.) and removed awaiting-review The author would like community review of the PR labels Aug 31, 2020
bors bot pushed a commit that referenced this pull request Aug 31, 2020
The definition of a `Scheme`, and the category of schemes as the full subcategory of locally ringed spaces.

Co-authored-by: Johan Commelin <johan@commelin.net>



Co-authored-by: Kevin Buzzard <k.buzzard@imperial.ac.uk>
Co-authored-by: Scott Morrison <scott.morrison@gmail.com>
Co-authored-by: Ashvni <ashvni.n@gmail.com>
@bors
Copy link

bors bot commented Aug 31, 2020

Pull request successfully merged into master.

Build succeeded:

@bors bors bot changed the title feature(algebraic_geometry/Scheme): the category of schemes [Merged by Bors] - feature(algebraic_geometry/Scheme): the category of schemes Aug 31, 2020
@bors bors bot closed this Aug 31, 2020
@bors bors bot deleted the LRS branch August 31, 2020 06:40
robertylewis pushed a commit that referenced this pull request Aug 31, 2020
The definition of a `Scheme`, and the category of schemes as the full subcategory of locally ringed spaces.

Co-authored-by: Johan Commelin <johan@commelin.net>



Co-authored-by: Kevin Buzzard <k.buzzard@imperial.ac.uk>
Co-authored-by: Scott Morrison <scott.morrison@gmail.com>
Co-authored-by: Ashvni <ashvni.n@gmail.com>
PatrickMassot pushed a commit that referenced this pull request Sep 8, 2020
The definition of a `Scheme`, and the category of schemes as the full subcategory of locally ringed spaces.

Co-authored-by: Johan Commelin <johan@commelin.net>



Co-authored-by: Kevin Buzzard <k.buzzard@imperial.ac.uk>
Co-authored-by: Scott Morrison <scott.morrison@gmail.com>
Co-authored-by: Ashvni <ashvni.n@gmail.com>
Sign up for free to subscribe to this conversation on GitHub. Already have an account? Sign in.
Labels
ready-to-merge All that is left is for bors to build and merge this PR. (Remember you need to say `bors r+`.)
Projects
None yet
Development

Successfully merging this pull request may close these issues.

7 participants