mathlib4 icon indicating copy to clipboard operation
mathlib4 copied to clipboard

feat(Algebra/Category/ModuleCat/Presheaf): the endofunctor of presheaves of modules induced by an oplax natural transformation

Open joelriou opened this issue 1 year ago • 2 comments

An endomorphism of ModuleCat.restrictScalarsPseudofunctor, i.e. a "compatible" family of functors ModuleCat R ⥤ ModuleCat R for all (commutative) rings R induces a functor PresheafOfModules R ⥤ PresheafOfModules R for any presheaf of (commutative) rings R. In particular, it should be possible to apply this to the exterior power functors in order to define the exterior powers of a presheaf of modules.


  • [ ] depends on: #18197

Open in Gitpod

joelriou avatar Oct 25 '24 16:10 joelriou

PR summary ea011743fb

Import changes for modified files

No significant changes to the import graph

Import changes for all files
Files Import difference
Mathlib.Algebra.Category.ModuleCat.Presheaf.FunctorOfNatTrans (new file) 1223

Declarations diff

+ CommRingCat.forgetToRingCat_map + CommRingCat.moduleCatRestrictScalarsPseudofunctor_mapComp' + CommRingCat.moduleCatRestrictScalarsPseudofunctor_mapId' + functorOfOplaxNatTrans + functorOfOplaxNatTransObj + mapComp' + mapComp'_eq_mapComp + mapId' + mapId'_eq_mapId + naturality_comp' + naturality_id'

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.


Increase in tech debt: (relative, absolute) = (1.05, 0.13)
Current number Change Type
845 6 erw
8 1 maxHeartBeats modifications

Current commit 61d8c488a0 Reference commit ea011743fb

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).

github-actions[bot] avatar Oct 25 '24 16:10 github-actions[bot]

This PR/issue depends on:

  • ~~leanprover-community/mathlib4#18197~~ By Dependent Issues (🤖). Happy coding!

I merged master to take a look at this, but it's now failing.

kim-em avatar Oct 28 '25 23:10 kim-em

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