Skip to content

Conversation

@joelriou
Copy link
Collaborator

@joelriou joelriou commented Oct 8, 2025

We define Scheme.Modules.pseudofunctor : Pseudofunctor (LocallyDiscrete Schemeᵒᵖ) (Adj Cat) which sends a scheme X to the category X.Modules of sheaves of modules (not to be be confused with the full subcategory of quasi-coherent sheaves). The target bicategory is the bicategory of adjunctions in the bicategory of categories: this means that we formalise both the pushforward and the pullback of sheaves of modules over schemes.


Open in Gitpod

@github-actions
Copy link

github-actions bot commented Oct 8, 2025

PR summary 337d737cae

Import changes for modified files

No significant changes to the import graph

Import changes for all files
Files Import difference

Declarations diff

+ Adjunction.toCat_id
+ Hom
+ Hom.toRingCatSheafHom
+ conjugateEquiv_eq_categoryTheoryConjugateEquiv
+ conjugateEquiv_leftAdjointCompIso_inv
+ conjugateEquiv_leftAdjointIdIso_hom
+ instance : Abelian X.Modules
+ instance : Category X.Modules
+ instance : Preadditive X.Modules
+ instance {X Y Z : Type*} [TopologicalSpace X] [TopologicalSpace Y] [TopologicalSpace Z]
+ mateEquiv_eq_categoryTheoryMateEquiv
+ ofCat
+ ofCat_toCat
+ pseudofunctor
+ pseudofunctor_associativity
+ pseudofunctor_left_unitality
+ pseudofunctor_right_unitality
+ pullback
+ pullbackComp
+ pullbackId
+ pullbackPushforwardAdjunction
+ pushforward
+ pushforwardComp
+ pushforwardId
+ toCat
+ toCat_comp_toCat
+ toCat_ofCat
++ conjugateEquiv_pullbackComp_inv
++ conjugateEquiv_pullbackId_hom
- instance : Abelian X.Modules := inferInstance
- instance : HasSheafify (Opens.grothendieckTopology X) AddCommGrpCat.{u}

You can run this locally as follows
## summary with just the declaration names:
./scripts/declarations_diff.sh <optional_commit>

## more verbose report:
./scripts/declarations_diff.sh long <optional_commit>

The doc-module for script/declarations_diff.sh contains some details about this script.


No changes to technical debt.

You can run this locally as

./scripts/technical-debt-metrics.sh pr_summary
  • The relative value is the weighted sum of the differences with weight given by the inverse of the current value of the statistic.
  • The absolute value is the relative value divided by the total sum of the inverses of the current values (i.e. the weighted average of the differences).

@mathlib4-dependent-issues-bot mathlib4-dependent-issues-bot added the blocked-by-other-PR This PR depends on another PR (this label is automatically managed by a bot) label Oct 8, 2025
@mathlib4-merge-conflict-bot mathlib4-merge-conflict-bot added the merge-conflict The PR has a merge conflict with master, and needs manual merging. (this label is managed by a bot) label Oct 12, 2025
@mathlib4-merge-conflict-bot
Copy link
Collaborator

This pull request has conflicts, please merge master and resolve them.

@github-actions github-actions bot removed the merge-conflict The PR has a merge conflict with master, and needs manual merging. (this label is managed by a bot) label Oct 30, 2025
@mathlib4-merge-conflict-bot mathlib4-merge-conflict-bot added the merge-conflict The PR has a merge conflict with master, and needs manual merging. (this label is managed by a bot) label Nov 19, 2025
@mathlib4-merge-conflict-bot
Copy link
Collaborator

This pull request has conflicts, please merge master and resolve them.

@mathlib4-dependent-issues-bot mathlib4-dependent-issues-bot removed the blocked-by-other-PR This PR depends on another PR (this label is automatically managed by a bot) label Nov 20, 2025
@joelriou joelriou added the WIP Work in progress label Nov 20, 2025
@github-actions github-actions bot removed merge-conflict The PR has a merge conflict with master, and needs manual merging. (this label is managed by a bot) large-import Automatically added label for PRs with a significant increase in transitive imports labels Nov 20, 2025
@joelriou joelriou removed the WIP Work in progress label Nov 21, 2025
Comment on lines +31 to +33
attribute [local simp] bicategoricalComp Cat.associator_hom_app Cat.associator_inv_app
Cat.leftUnitor_hom_app Cat.leftUnitor_inv_app Cat.rightUnitor_hom_app Cat.rightUnitor_inv_app
Functor.toCatHom
Copy link
Member

Choose a reason for hiding this comment

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

Should this be a simp set?

Comment on lines +38 to +49
abbrev toCat : Bicategory.Adjunction F.toCatHom G.toCatHom where
unit := adj.unit
counit := adj.counit

/-- The adjunction of functors corresponding to an adjunction in the bicategory `Cat`. -/
abbrev ofCat {C D : Cat} {F : C ⟶ D} {G : D ⟶ C}
(adj : Bicategory.Adjunction F G) :
Functor.ofCatHom F ⊣ Functor.ofCatHom G where
unit := adj.unit
counit := adj.counit
left_triangle_components X := by simpa using congr_app adj.left_triangle X
right_triangle_components X := by simpa using congr_app adj.right_triangle X
Copy link
Member

Choose a reason for hiding this comment

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

Why are these abbrevs?

namespace Bicategory

@[simp]
lemma Adjunction.toCat_id (C : Cat.{v, u}) :
Copy link
Member

Choose a reason for hiding this comment

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

Suggested change
lemma Adjunction.toCat_id (C : Cat.{v, u}) :
lemma Adjunction.ofCat_id (C : Cat.{v, u}) :

Comment on lines +15 to +17
and show that the left adjoint functors satisfies properties similar to the left/right
unitality and the associativity of pseudofunctors if the right adjoint functors
satisfy the corresponding properties.
satisfies the corresponding properties.
Copy link
Member

Choose a reason for hiding this comment

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

I think satisfy was correct?

Comment on lines +173 to +176
attribute [simps! obj_obj map_l map_r map_adj] pseudofunctor
attribute [simps! mapId_hom_τl mapId_hom_τr mapId_inv_τl mapId_inv_τr] pseudofunctor
attribute [simps! mapComp_hom_τl mapComp_hom_τr] pseudofunctor
attribute [simps! mapComp_inv_τl mapComp_inv_τr] pseudofunctor
Copy link
Member

Choose a reason for hiding this comment

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

Why are these done separately? Is it because it times out otherwise?

@erdOne erdOne added the awaiting-author A reviewer has asked the author a question or requested changes. label Nov 21, 2025
Comment on lines +33 to +37
/-- The morphism of sheaves of rings corresponding to a morphism of schemes. -/
def Hom.toRingCatSheafHom (f : X ⟶ Y) :
Y.ringCatSheaf ⟶ ((TopologicalSpace.Opens.map f.base).sheafPushforwardContinuous
_ _ _).obj X.ringCatSheaf where
val := Functor.whiskerRight f.c _
Copy link
Member

Choose a reason for hiding this comment

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

I think this should go near Scheme.ringCatSheaf

Sign up for free to join this conversation on GitHub. Already have an account? Sign in to comment

Labels

awaiting-author A reviewer has asked the author a question or requested changes. t-algebraic-geometry Algebraic geometry

Projects

None yet

Development

Successfully merging this pull request may close these issues.

4 participants