mathlib4
mathlib4 copied to clipboard
feat(Bicategory/Functorbicategory): define bicategory of pseudofunctors
This PR contains a definition of the bicategory of pseudofunctors, in the file Bicategory/FunctorBicategory/Pseudo.lean. It also moves the file Bicategory/Functorbicategory.lean to Bicategory/FunctorBicategory/Oplax.lean.
- [x] depends on: #14028
- [ ] depends on: #18250
- [ ] depends on: #18252
- [ ] depends on: #18253
PR summary 77c1deedba
Import changes for modified files
No significant changes to the import graph
Import changes for all files
| Files | Import difference |
|---|---|
Mathlib.CategoryTheory.Bicategory.Modification.Pseudo (new file) |
359 |
Mathlib.CategoryTheory.Bicategory.FunctorBicategory.Pseudo (new file) |
361 |
Declarations diff
+ associator
+ bicategory
+ leftUnitor
+ rightUnitor
+ whiskerLeft
+ whiskerRight
++ ModificationIso.ofComponents
++ equivOplax
++ hasCoeToOplax
++ mkOfOplax
++ toOplax
++ whiskerLeft_naturality
++ whiskerRight_naturality
+++ homCategory.ext
- Modification.comp_app'
- Modification.id_app'
- ext
- id
- vcomp
-+++ Modification
-+++ instance : Inhabited (Modification η η)
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
relativevalue is the weighted sum of the differences with weight given by the inverse of the current value of the statistic. - The
absolutevalue is therelativevalue divided by the total sum of the inverses of the current values (i.e. the weighted average of the differences).
This PR/issue depends on:
- ~~leanprover-community/mathlib4#14028~~
- ~~leanprover-community/mathlib4#18250~~
- ~~leanprover-community/mathlib4#18252~~
- ~~leanprover-community/mathlib4#18253~~
- leanprover-community/mathlib4#18254 By Dependent Issues (🤖). Happy coding!
Now that I have added Lax functors, I think this should be rewritten so that Strong natural transformations of Pseudofunctors are not defined to be strong natural tranformations of the underlying oplax functors. I'm not sure when I plan to get around to this.
This pull request has conflicts, please merge master and resolve them.
This pull request has conflicts, please merge master and resolve them.
This pull request has conflicts, please merge master and resolve them.