Skip to content

Conversation

joelriou
Copy link
Collaborator

@joelriou joelriou commented Jun 24, 2025

In this PR, we formalize an existence theorem for right derived functors which appeared in the article Structures de dérivabilité by Bruno Kahn and Georges Maltsiniotis, Adv. Math. 218 (2008).


This PR continues the work from #22508.

Original PR: #22508

@joelriou
Copy link
Collaborator Author

Comments from Original PR #22508

This section contains 1 comment(s) from the original PR, excluding bot comments.


@github-actions (2025-03-03 17:04 UTC):

PR summary 5d11a5f926

Import changes for modified files

No significant changes to the import graph

Import changes for all files
Files Import difference
Mathlib.CategoryTheory.Functor.Derived.PointwiseRightDerived (new file) 474
Mathlib.CategoryTheory.Localization.DerivabilityStructure.PointwiseRightDerived (new file) 643

Declarations diff

+ HasPointwiseRightDerivedFunctor
+ HasPointwiseRightDerivedFunctorAt
+ LeftExtension.isPointwiseLeftKanExtensionOfIsIso
+ hasColimit_comp_iff
+ hasLimit_comp_iff
+ hasLimit_equivalence_comp
+ hasLimit_of_equivalence_comp
+ hasPointwiseLeftKanExtensionAt_iff_of_equivalence
+ hasPointwiseLeftKanExtensionAt_iff_of_iso
+ hasPointwiseLeftKanExtensionAt_iff_of_iso'
+ hasPointwiseLeftKanExtensionAt_of_equivalence
+ hasPointwiseLeftKanExtension_of_hasPointwiseRightDerivedFunctor
+ hasPointwiseRightDerivedFunctorAt_iff
+ hasPointwiseRightDerivedFunctorAt_iff_of_isRightDerivabilityStructure
+ hasPointwiseRightDerivedFunctorAt_iff_of_mem
+ hasPointwiseRightDerivedFunctor_iff_of_isRightDerivabilityStructure
+ hasPointwiseRightDerivedFunctor_of_inverts
+ hasPointwiseRightKanExtensionAt_iff_of_equivalence
+ hasPointwiseRightKanExtensionAt_iff_of_iso
+ hasPointwiseRightKanExtensionAt_iff_of_iso'
+ hasPointwiseRightKanExtensionAt_of_equivalence
+ hasRightDerivedFunctor_of_hasPointwiseRightDerivedFunctor
+ instance :
+ isIso_comp_left_iff
+ isIso_comp_right_iff
+ isIso_α_iff_of_isRightDerivabilityStructure
+ isPointwiseLeftKanExtensionAtEquivOfIso'
+ isPointwiseLeftKanExtensionAtOfIso
+ isPointwiseLeftKanExtensionAtOfIso'
+ isPointwiseLeftKanExtensionOfHasPointwiseRightDerivedFunctor
+ isPointwiseLeftKanExtensionOfIso
+ isPointwiseRightKanExtensionAtEquivOfIso'
+ isPointwiseRightKanExtensionAtOfIso'
+ rightDerivedFunctorComparison
+ rightDerivedFunctorComparison_fac
+ rightDerivedFunctorComparison_fac_app

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

@github-actions github-actions bot added merge-conflict The PR has a merge conflict with master, and needs manual merging. (this label is managed by a bot) t-category-theory Category theory labels Jun 24, 2025
@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 Jun 24, 2025
…nctor' into jriou-derivability-structure-pointwise
@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 Jun 24, 2025
Copy link

github-actions bot commented Jun 24, 2025

PR summary cc0d5cbbe4

Import changes for modified files

No significant changes to the import graph

Import changes for all files
Files Import difference
Mathlib.CategoryTheory.GuitartExact.KanExtension (new file) 638
Mathlib.CategoryTheory.Localization.DerivabilityStructure.PointwiseRightDerived (new file) 679

Declarations diff

+ IsPointwiseLeftKanExtension.compTwoSquare
+ compTwoSquare
+ hasColimit_comp_iff
+ hasLeftKanExtension
+ hasLimit_comp_iff
+ hasPointwiseLeftKanExtension
+ hasPointwiseLeftKanExtensionAt_iff
+ hasPointwiseLeftKanExtension_iff
+ hasPointwiseRightDerivedFunctorAt_iff_of_isRightDerivabilityStructure
+ hasPointwiseRightDerivedFunctor_iff_of_isRightDerivabilityStructure
+ instance (Y : D) : Subsingleton (E.IsPointwiseLeftKanExtensionAt Y)
+ instance (Y : D) : Subsingleton (E.IsPointwiseRightKanExtensionAt Y)
+ instance : IsIso (Φ.rightDerivedFunctorComparison L₁ L₂ F F₁ α₁ F₂ α₂) := by
+ isIso_comp_left_iff
+ isIso_comp_right_iff
+ isIso_α_iff_of_isRightDerivabilityStructure
+ isPointwiseLeftKanExtensionAtCompTwoSquareEquiv
+ isPointwiseLeftKanExtensionEquivOfGuitartExact
+ isPointwiseLeftKanExtensionOfCompTwoSquare
+ nonempty_isPointwiseLeftKanExtensionAt_compTwoSquare_iff
+ rightDerivedFunctorComparison
+ rightDerivedFunctorComparison_fac
+ rightDerivedFunctorComparison_fac_app

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

@leanprover-community-bot-assistant leanprover-community-bot-assistant added the merge-conflict The PR has a merge conflict with master, and needs manual merging. (this label is managed by a bot) label Jul 11, 2025
@leanprover-community-bot-assistant
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 Aug 13, 2025
@mathlib4-dependent-issues-bot
Copy link
Collaborator

mathlib4-dependent-issues-bot commented Aug 13, 2025

@joelriou joelriou added the WIP Work in progress label Aug 13, 2025
@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 5, 2025
@joelriou joelriou added WIP Work in progress and removed WIP Work in progress labels Oct 5, 2025
@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 9, 2025
Sign up for free to join this conversation on GitHub. Already have an account? Sign in to comment

Labels

blocked-by-other-PR This PR depends on another PR (this label is automatically managed by a bot) t-category-theory Category theory WIP Work in progress

Projects

None yet

Development

Successfully merging this pull request may close these issues.

3 participants