mathlib4 icon indicating copy to clipboard operation
mathlib4 copied to clipboard

feat(CategoryTheory): right derived functors

Open joelriou opened this issue 1 year ago • 1 comments

In this PR, given a functor F : C ⥤ H, and L : C ⥤ D that is a localization functor for W : MorphismProperty C, we define F.totalRightDerived L W : D ⥤ H as the left Kan extension of F along L: it is defined if the type class F.HasRightDerivedFunctor W asserting the existence of a left Kan extension is satisfied.


  • [x] depends on: #12785

Open in Gitpod

joelriou avatar May 09 '24 15:05 joelriou

This PR/issue depends on:

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

Do we have left derived functors yet? Thanks Joël and Dagur maintainer merge

erdOne avatar Jun 05 '24 09:06 erdOne

🚀 Pull request has been placed on the maintainer queue by erdOne.

github-actions[bot] avatar Jun 05 '24 09:06 github-actions[bot]

How does this mesh with Mathlib/CategoryTheory/Abelian/RightDerived.lean?

jcommelin avatar Jun 05 '24 09:06 jcommelin

How does this mesh with Mathlib/CategoryTheory/Abelian/RightDerived.lean?

Eventually, Abelian.RightDerived will be refactored (as in my draft branch https://github.com/leanprover-community/mathlib4/blob/jriou_localization/Mathlib/Algebra/Homology/DerivedCategory/RightDerivedFunctorPlus.lean#L207 ), but we need more material: derived categories, the injective derivability structure, existence of derived functors from derivability structures, etc.

Do we have left derived functors yet?

No, but I would rather develop the right side more before dualising the results.

joelriou avatar Jun 05 '24 09:06 joelriou

How does this mesh with Mathlib/CategoryTheory/Abelian/RightDerived.lean?

Eventually, Abelian.RightDerived will be refactored (as in my draft branch https://github.com/leanprover-community/mathlib4/blob/jriou_localization/Mathlib/Algebra/Homology/DerivedCategory/RightDerivedFunctorPlus.lean#L207 ), but we need more material: derived categories, the injective derivability structure, existence of derived functors from derivability structures, etc.

@joelriou could you please explain this in a comment in both files? Then people can be aware of the dual development of the theory for the time being.

jcommelin avatar Jun 05 '24 10:06 jcommelin

@joelriou could you please explain this in a comment in both files? Then people can be aware of the dual development of the theory for the time being.

Thanks for the suggestion. I have just added TODO in the relevant files.

joelriou avatar Jun 05 '24 11:06 joelriou

Thanks :tada:

bors merge

jcommelin avatar Jun 05 '24 11:06 jcommelin

Pull request successfully merged into master.

Build succeeded:

mathlib-bors[bot] avatar Jun 05 '24 13:06 mathlib-bors[bot]