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

feat(topology/sheaves/Godement): define the first term of Godement resolution #16878

Draft
wants to merge 9 commits into
base: master
Choose a base branch
from

Conversation

jjaassoonn
Copy link
Collaborator


Open in Gitpod

@jjaassoonn jjaassoonn added awaiting-review The author would like community review of the PR awaiting-CI The author would like to see what CI has to say before doing more work. t-algebraic-geometry Algebraic geometry labels Oct 9, 2022
@github-actions github-actions bot removed the awaiting-CI The author would like to see what CI has to say before doing more work. label Oct 9, 2022
Under the isomorphism `godement_presheaf(𝓕, U) ≅ ∏ₓ skyscraper(x, 𝓕ₓ)(U)`, there is a morphism
`𝓕 ⟶ ∏ₓ skyscraper(x, 𝓕ₓ) ≅ godement_presheaf(𝓕)`
-/
@[simps] def to_godement_presheaf : 𝓕 ⟶ godement_presheaf 𝓕 :=
Copy link
Collaborator

Choose a reason for hiding this comment

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

Would it be easier to work with the definition

def to_godement_presheaf : 𝓕 ⟶ godement_presheaf 𝓕 :=
pi.lift $ λ p₀, (stalk_skyscraper_presheaf_adjunction_auxs.unit p₀).app 𝓕

? I guess it depends on what you want to do with it?

Copy link
Collaborator Author

Choose a reason for hiding this comment

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

This definition is certainly more concise. All I need from this definition is this lemma, which should also hold for your definition modulo some modification. So I will use your definition instead.

Copy link
Collaborator

Choose a reason for hiding this comment

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

I mentioned this to you a while ago but maybe you didn't notice :)

@jjaassoonn jjaassoonn added awaiting-author A reviewer has asked the author a question or requested changes and removed awaiting-review The author would like community review of the PR labels Oct 9, 2022
universes u v

variables {X : Top.{u}} {C : Type u} [category.{u} C]
variables [has_limits C] [has_terminal C] [has_colimits C]
Copy link
Collaborator

Choose a reason for hiding this comment

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

Suggested change
variables [has_limits C] [has_terminal C] [has_colimits C]
variables [has_limits C] [has_colimits C]

has_limits implieshas_terminal.

Copy link
Collaborator

@alreadydone alreadydone Oct 9, 2022

Choose a reason for hiding this comment

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

Actually, has_products suffice for this file, right? But we lack an instance from has_products to has_terminal. Maybe has_products_of_shape X + has_terminal?

We have category_theory.limits.functor_category_has_limits_of_shape but since presheaf is not a reducible def we need to manually add one more instance to topology/sheaves/limits for Lean to infer that the presheaf category also has limits of shape X.

Copy link
Collaborator Author

Choose a reason for hiding this comment

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

we still need has_colimits C for stalks

Copy link
Member

Choose a reason for hiding this comment

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

You should only need has_filtered_colimits for that, right?

Copy link
Collaborator Author

Choose a reason for hiding this comment

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

stalk_functor assumes has_colimits, so has_colimits cannot be relaxed

Copy link
Collaborator Author

Choose a reason for hiding this comment

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

Actually, has_products suffice for this file, right? But we lack an instance from has_products to has_terminal. Maybe has_products_of_shape X + has_terminal?

We have category_theory.limits.functor_category_has_limits_of_shape but since presheaf is not a reducible def we need to manually add one more instance to topology/sheaves/limits for Lean to infer that the presheaf category also has limits of shape X.

limit_is_sheaf requires has_limits C

@jjaassoonn jjaassoonn requested a review from a team as a code owner October 11, 2022 13:31
@jjaassoonn jjaassoonn added awaiting-review The author would like community review of the PR awaiting-CI The author would like to see what CI has to say before doing more work. and removed awaiting-author A reviewer has asked the author a question or requested changes labels Oct 11, 2022
@jjaassoonn jjaassoonn marked this pull request as draft May 8, 2023 15:53
@kim-em kim-em added the too-late This PR was ready too late for inclusion in mathlib3 label Jul 16, 2023
@kim-em kim-em removed the request for review from a team August 6, 2023 09:58
Sign up for free to subscribe to this conversation on GitHub. Already have an account? Sign in.
Labels
awaiting-CI The author would like to see what CI has to say before doing more work. awaiting-review The author would like community review of the PR t-algebraic-geometry Algebraic geometry too-late This PR was ready too late for inclusion in mathlib3
Projects
None yet
Development

Successfully merging this pull request may close these issues.

4 participants