mathlib4
mathlib4 copied to clipboard
The math library of Lean 4
--- [](https://gitpod.io/from-referrer/)
--- [](https://gitpod.io/from-referrer/)
--- Preliminary to removing the order dependency from `Mathlib/Data/Nat/Defs.lean`, but that needs a little more work [](https://gitpod.io/from-referrer/)
In characteristic zero, a [semisimple Lie algebra](https://leanprover-community.github.io/mathlib4_docs/Mathlib/Algebra/Lie/Semisimple.html#LieAlgebra.IsSemisimple) is a direct sum of [simple Lie algebra](https://leanprover-community.github.io/mathlib4_docs/Mathlib/Algebra/Lie/Semisimple.html#LieAlgebra.IsSimple)s. We should add this result to Mathlib. I think the most useful statement of this...
testing more aggressive caching --- [](https://gitpod.io/from-referrer/)
Show `Gamma'(1/2) = -√π * (γ + 2 * log 2)` and various other related results. --- [](https://gitpod.io/from-referrer/)
--- [](https://gitpod.io/from-referrer/)
--- [](https://gitpod.io/from-referrer/)
This PR creates the file `CategoryTheory.Sites.LocallyInjective` which develops the basic API of locally injective morphisms of presheaves. The file `CategoryTheory.Sites.Surjective` is renamed `CategoryTheory.Sites.LocallySurjective` and shall be expanded in a future...
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...