Welcome to the mathlib review page. Everybody's help with reviewing is appreciated. Reviewing contributions is important, and everybody is welcome to review pull requests! If you're not sure how, the pull request review guide is there to help you.
This page contains tables of
Number |
Author |
Title |
Description |
Labels |
+/- |
Modified files (first 100) |
📝 |
💬 |
All users who commented or reviewed |
Assignee(s) |
Updated |
Last status change |
total time in review |
20719 |
gio256 author:gio256 |
feat(AlgebraicTopology): delaborators for truncated simplicial notations |
We add delaborators for the following notations, introduced in #20688:
- `⦋m⦌ₙ`, which denotes the `m`-dimensional simplex in the `n`-truncated simplex category.
- `X _⦋m⦌ₙ`, which denotes the `m`-th term of an `n`-truncated simplicial object `X`.
- `X ^⦋m⦌ₙ`, which denotes the `m`-th term of an `n`-truncated cosimplicial object `X`.
If `pp.proofs` is set to `true`, we also pretty-print the proof `p : m ≤ n` for all three notations as `⦋m, p⦌ₙ`, `X _⦋m, p⦌ₙ`, and `X ^⦋m, p⦌ₙ`, respectively.
Credit to @kmill for one piece of code and much metaprogramming inspiration.
---
- [x] depends on: #20688
- [x] depends on: #23018
[](https://gitpod.io/from-referrer/)
|
infinity-cosmos
t-category-theory
t-meta
|
525/33 |
Mathlib.lean,Mathlib/AlgebraicTopology/SimplexCategory/Basic.lean,Mathlib/AlgebraicTopology/SimplexCategory/Defs.lean,Mathlib/AlgebraicTopology/SimplicialObject/Basic.lean,Mathlib/Tactic.lean,Mathlib/Tactic/SimplexCategory.lean,Mathlib/Util/Superscript.lean,MathlibTest/SimplexCategory.lean,MathlibTest/SimplicialObject.lean,MathlibTest/superscript.lean,scripts/noshake.json |
11 |
22 |
['eric-wieser', 'gio256', 'github-actions', 'kim-em', 'mathlib4-dependent-issues-bot'] |
eric-wieser assignee:eric-wieser |
79-36528 2 months ago |
79-39169 2 months ago |
88-24308 88 days |
24266 |
plp127 author:plp127 |
feat(Order): `NoBotOrder α` implies `NoMinOrder α` under `IsDirected α (· ≥ ·)` |
Proves that `NoBotOrder α` implies `NoMinOrder α` under `IsDirected α (· ≥ ·)`, and also the dual theorem.
---
[](https://gitpod.io/from-referrer/)
|
t-order |
14/0 |
Mathlib/Order/Directed.lean |
1 |
4 |
['github-actions', 'plp127', 'urkud'] |
nobody |
78-6011 2 months ago |
89-17392 2 months ago |
89-17373 89 days |
22231 |
pechersky author:pechersky |
feat(Algebra/Valued): `AdicExpansion` initial defns |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-topology
label:t-algebra$ |
299/0 |
Mathlib.lean,Mathlib/Topology/Algebra/Valued/AdicExpansion.lean |
2 |
2 |
['Thmoas-Guan', 'github-actions'] |
nobody |
77-2770 2 months ago |
146-4412 4 months ago |
146-4534 146 days |
22464 |
adomani author:adomani |
feat(CI): declarations diff in Lean |
Rewrites the `declaration_diff` script in Lean.
You can see the effect of the new script in the testing branch #22497.
The new CI step runs in approximately 5mins, but is separate from the `build` step.
---
[](https://gitpod.io/from-referrer/)
|
CI |
151/0 |
.github/workflows/PR_summary_lean.yml,scripts/README.md,scripts/declarations_diff.lean,scripts/declarations_diff_lean_shell_glue.sh |
4 |
6 |
['bryangingechen', 'github-actions', 'grunweg'] |
robertylewis assignee:robertylewis |
72-76108 2 months ago |
137-40353 4 months ago |
137-40339 137 days |
23758 |
erdOne author:erdOne |
feat(Topology/Algebra): linearly topologized iff non-archimedian |
...for topological modules over compact rings or `ℤ`-finite rings
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebra
t-topology
label:t-algebra$ |
138/3 |
Mathlib/LinearAlgebra/Span/Basic.lean,Mathlib/Topology/Algebra/LinearTopology.lean |
2 |
21 |
['ADedecker', 'AntoineChambert-Loir', 'erdOne', 'github-actions', 'grunweg'] |
ADedecker and AntoineChambert-Loir assignee:AntoineChambert-Loir assignee:ADedecker |
72-55580 2 months ago |
93-28024 3 months ago |
103-76839 103 days |
22196 |
xyzw12345 author:xyzw12345 |
feat: `lie_ring` tactic and `LieReduce` command |
In this PR, we implement a new tactic that reduces expressions in a `LieRing` to a normal form and checks whether they are equal, and a command which reduces the expression and displays the normal form.
The implementation of this tactic imitates the `ring` tactic, using the `Qq` package to implement a specific reduction algorithm, following the theory of Hall sets and Lyndon words. A reference for the algorithm can be found at, for example, [here](https://personal.math.ubc.ca/~cass/research/pdf/Free.pdf).
This project is the result of a workshop at Peking University, and @siddhartha-gadgil has helped us a lot on understanding the concepts in metaprogramming.
Edit: The changes are reverted to a point where only `AtomM` is used.
Co-authored-by:
@Thmoas-Guan <2300010733@stu.pku.edu.cn>
@yhtq <2100012990@stu.pku.edu.cn>
@Blackfeather007 <2100017455@stu.pku.edu.cn>
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-meta
|
816/2 |
Mathlib.lean,Mathlib/Algebra/Lie/Derivation/AdjointAction.lean,Mathlib/Tactic.lean,Mathlib/Tactic/LieAlgebra/Basic.lean,Mathlib/Tactic/LieAlgebra/LieRingNF.lean,Mathlib/Util/AtomM.lean,MathlibTest/lie_ring.lean,scripts/noshake.json |
8 |
16 |
['bryangingechen', 'eric-wieser', 'faenuccio', 'github-actions', 'grunweg', 'ocfnash', 'siddhartha-gadgil', 'xyzw12345'] |
robertylewis assignee:robertylewis |
71-59443 2 months ago |
147-4542 4 months ago |
147-4530 147 days |
24602 |
xyzw12345 author:xyzw12345 |
feat(LinearAlgebra/SymmetricAlgebra): IsSymmetricAlgebra |
This PR is a part of #21539, which separates out the part about `IsSymmetricAlgebra`.
Co-authored-by: Raphael Douglas Giles @Raph-DG
Co-authored-by: Zhixuan Dai <22300180006@m.fudan.edu.cn>
Co-authored-by: Zhenyan Fu
Co-authored-by: Yiming Fu
- [ ] depends on: #21539
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
78/0 |
Mathlib/LinearAlgebra/SymmetricAlgebra/Basic.lean,Mathlib/LinearAlgebra/SymmetricAlgebra/Basis.lean |
2 |
5 |
['eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
69-41336 2 months ago |
69-41588 2 months ago |
69-43526 69 days |
23238 |
YaelDillies author:YaelDillies |
feat: extended floor and ceil |
My motivation for this is to prove `ENat.toENNReal (⨆ i, f i) = ⨆ i, ENat.toENNReal (f i)` and `ENat.toENNReal (⨅ i, f i) = ⨅ i, ENat.toENNReal (f i)`. Kalle Kytölä independently needs this for his formalisation of statistical physics.
From MiscYD
---
- [x] depends on: #24781
- [x] depends on: #24782
See #15269 for a past attempt.
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
235/0 |
Mathlib.lean,Mathlib/Algebra/Order/Floor/Extended.lean |
2 |
24 |
['YaelDillies', 'b-mehta', 'eric-wieser', 'github-actions', 'kkytola', 'mathlib4-dependent-issues-bot', 'urkud'] |
nobody |
69-30744 2 months ago |
69-36695 2 months ago |
117-2513 117 days |
24184 |
YaelDillies author:YaelDillies |
feat: `[G : H]` notation for the index of `H : Subgroup G` |
This is a cute notation which I wrote for FLT. Not sure whether we want it in mathlib nor how to include `relindex` in the picture.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
RFC
label:t-algebra$ |
5/0 |
Mathlib/GroupTheory/Index.lean |
1 |
7 |
['YaelDillies', 'erdOne', 'github-actions', 'j-loreaux', 'kbuzzard'] |
nobody |
69-737 2 months ago |
69-737 2 months ago |
92-24854 92 days |
24829 |
urkud author:urkud |
fix(Topology/Homotopy): fix name&args order of `comp` |
`ContinuousMap.Homotopy.hcomp` used name & arguments order
that matches Mathlib's category theory conventions,
not topology conventions.
---
[](https://gitpod.io/from-referrer/)
|
t-topology |
30/19 |
Mathlib/Topology/Homotopy/Basic.lean,Mathlib/Topology/Homotopy/Contractible.lean,Mathlib/Topology/Homotopy/Equiv.lean,Mathlib/Topology/Homotopy/Lifting.lean |
4 |
5 |
['github-actions', 'grunweg', 'urkud'] |
nobody |
67-77252 2 months ago |
67-85892 2 months ago |
67-85943 67 days |
24752 |
MichaelStollBayreuth author:MichaelStollBayreuth |
perf(Data.Real.Sqrt): make Real.sqrt irreducible |
We try to see what happens if we make `Real.sqrt` irreducible.
There are cases where this makes unification *very* significantly faster, compare [#mathlib4 > Coercion triggers timeout @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Coercion.20triggers.20timeout/near/517177117).
---
[](https://gitpod.io/from-referrer/)
|
t-data |
1/0 |
Mathlib/Data/Real/Sqrt.lean |
1 |
18 |
['MichaelStollBayreuth', 'eric-wieser', 'github-actions', 'leanprover-bot'] |
nobody |
67-33179 2 months ago |
69-46501 2 months ago |
69-51975 69 days |
24870 |
smmercuri author:smmercuri |
feat: `Field`, `FiniteDimensional` and `Algebra.IsSeparable` instances for `WithAbs` |
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-analysis
|
14/1 |
Mathlib/Analysis/Normed/Field/WithAbs.lean |
1 |
1 |
['github-actions'] |
nobody |
66-78634 2 months ago |
66-78641 2 months ago |
66-78782 66 days |
24872 |
smmercuri author:smmercuri |
feat: `apply` and `coe` results for `UniformSpace.Completion.mapRingHom` |
---
[](https://gitpod.io/from-referrer/)
|
t-topology |
9/0 |
Mathlib/Topology/Algebra/UniformRing.lean |
1 |
1 |
['github-actions'] |
nobody |
66-78413 2 months ago |
66-78413 2 months ago |
66-78458 66 days |
24889 |
Kha author:Kha |
chore: do not include cache requests in build benchmark |
|
|
5/2 |
scripts/bench/temci-config.run.yml |
1 |
4 |
['Kha', 'github-actions', 'leanprover-bot'] |
nobody |
66-58627 2 months ago |
66-68462 2 months ago |
66-68442 66 days |
24311 |
YaelDillies author:YaelDillies |
chore: replace `Monoid.IsTorsionFree` with `IsMulTorsionFree` |
From Toric
---
- [x] depends on: #24312
[](https://gitpod.io/from-referrer/)
|
toric
t-algebra
label:t-algebra$ |
63/29 |
Mathlib/Algebra/Group/Torsion.lean,Mathlib/Combinatorics/Additive/CauchyDavenport.lean,Mathlib/GroupTheory/Order/Min.lean,Mathlib/GroupTheory/Torsion.lean,Mathlib/Topology/Instances/ZMultiples.lean |
5 |
5 |
['YaelDillies', 'b-mehta', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
66-53782 2 months ago |
66-53782 2 months ago |
66-67109 66 days |
22043 |
YaelDillies author:YaelDillies |
chore: shortcut instance for `Neg ℤˣ` |
This lets us avoid importing `Ring` in downstream files (most of the effect is to come).
---
[](https://gitpod.io/from-referrer/)
|
file-removed
t-algebra
label:t-algebra$ |
20/47 |
Mathlib.lean,Mathlib/Algebra/GCDMonoid/Nat.lean,Mathlib/Algebra/Group/Int/Units.lean,Mathlib/Algebra/Order/Ring/Abs.lean,Mathlib/Algebra/Ring/Int/Units.lean,Mathlib/Algebra/Ring/NegOnePow.lean,Mathlib/Data/Fintype/Units.lean,Mathlib/Data/Int/AbsoluteValue.lean,Mathlib/Data/Int/Associated.lean,Mathlib/GroupTheory/HNNExtension.lean,Mathlib/NumberTheory/NumberField/Basic.lean,MathlibTest/Zify.lean |
12 |
15 |
['YaelDillies', 'eric-wieser', 'github-actions', 'j-loreaux', 'leanprover-community-bot-assistant', 'mathlib-bors'] |
nobody |
66-53525 2 months ago |
66-53525 2 months ago |
151-26558 151 days |
24891 |
YaelDillies author:YaelDillies |
feat: `M ≃ₗ[R] (Fin (Module.finrank R M) → R)` for `M` a finite `R`-module |
From Toric
---
[](https://gitpod.io/from-referrer/)
|
toric
t-algebra
label:t-algebra$ |
13/3 |
Mathlib/LinearAlgebra/Dimension/Free.lean,Mathlib/LinearAlgebra/FreeModule/Basic.lean,Mathlib/LinearAlgebra/FreeModule/Finite/Basic.lean |
3 |
9 |
['YaelDillies', 'erdOne', 'eric-wieser', 'github-actions'] |
nobody |
65-40629 2 months ago |
66-50460 2 months ago |
66-67379 66 days |
24533 |
robertmaxton42 author:robertmaxton42 |
feat (ULift): conjugation by ULift.up/down, misc cast/heq lemmas |
* Adds the convenience def `ULift.conj x := `down (f (up x))`, and corresponding basic lemmas
* Adds lemmas showing that `ULift.up` and `.down` commute with casts and preserve `HEq`.
---
[](https://gitpod.io/from-referrer/)
|
t-data |
31/0 |
Mathlib/Data/ULift.lean |
1 |
14 |
['eric-wieser', 'github-actions', 'robertmaxton42'] |
nobody |
62-68205 2 months ago |
78-67845 2 months ago |
78-75757 78 days |
22300 |
chrisflav author:chrisflav |
feat(RingTheory/GoingDown): lift `LTSeries` of primes |
Inductive version of `Ideal.exists_ideal_lt_liesOver_of_lt`.
Co-authored by: Sihan Su
Co-authored by: Yi Song
---
- [x] depends on: #22299
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
27/0 |
Mathlib/RingTheory/Ideal/GoingDown.lean |
1 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
61-39001 2 months ago |
61-39125 2 months ago |
61-42587 61 days |
25044 |
alreadydone author:alreadydone |
feat(Topology/Algebra): `Homeomorph` version of `unitsEquivNeZero` |
also add `Topology.IsEmbedding.homeomorphImage`: a set is homeomorphic to its image under any embedding.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-topology
label:t-algebra$ |
51/28 |
Mathlib/Topology/Algebra/GroupWithZero.lean,Mathlib/Topology/Homeomorph/Lemmas.lean |
2 |
1 |
['github-actions'] |
nobody |
60-57404 1 month ago |
60-61659 1 month ago |
60-61641 60 days |
24333 |
xcloudyunx author:xcloudyunx |
feat(Combinatorics/SimpleGraph): cycle graph implementation for generic vertex types |
The existing `cycleGraph` implementation under Combinatorics/SimpleGraph/Circulant.lean only operates over `Fin n`. This PR implements a cycle graph implementation over any generic vertex type.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-combinatorics
|
187/0 |
Mathlib.lean,Mathlib/Combinatorics/SimpleGraph/Cycle.lean |
2 |
29 |
['IvanRenison', 'github-actions'] |
kmill assignee:kmill |
59-11222 1 month ago |
87-8779 2 months ago |
87-8830 87 days |
25123 |
eric-wieser author:eric-wieser |
feat: add rfl lemmas for monoidal categories |
Making these `simp` opens a can of worms best left to #24823
`simps` would generate bad names here.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
111/0 |
Mathlib/Algebra/Category/AlgCat/Monoidal.lean,Mathlib/Algebra/Category/ModuleCat/Monoidal/Basic.lean,Mathlib/LinearAlgebra/QuadraticForm/QuadraticModuleCat/Monoidal.lean |
3 |
1 |
['github-actions'] |
nobody |
58-11029 1 month ago |
58-11029 1 month ago |
58-11080 58 days |
24528 |
chrisflav author:chrisflav |
feat(AlgebraicGeometry): directed covers |
Directed covers are covers, where every intersection can be covered by a component of the cover. For open covers this is equivalent to the images forming a basis of the topology.
If a cover is directed, the compatibility conditions for gluing become easier, because only compatibility with the transition maps needs to be checked.
---
[](https://gitpod.io/from-referrer/)
|
t-algebraic-geometry |
233/0 |
Mathlib.lean,Mathlib/AlgebraicGeometry/Cover/Directed.lean |
2 |
6 |
['chrisflav', 'erdOne', 'github-actions', 'joelriou', 'leanprover-community-bot-assistant'] |
nobody |
57-54895 1 month ago |
57-54962 1 month ago |
74-39983 74 days |
25069 |
erdOne author:erdOne |
feat(EllipticCurve): rational points of singular nodal cubics |
---
[](https://gitpod.io/from-referrer/)
|
t-algebraic-geometry |
251/0 |
Mathlib.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Affine/Basic.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Singular/Node.lean |
3 |
11 |
['Multramate', 'acmepjz', 'erdOne', 'github-actions'] |
nobody |
57-46235 1 month ago |
60-6737 1 month ago |
60-6792 60 days |
24050 |
Paul-Lez author:Paul-Lez |
feat(Data/Finsupp/Pointwise): generalise pointwise scalar multiplication of finsupps |
As pointed out by @eric-wieser, this creates an instance diamond with `SMul (α → β) (α →₀ (α → β))`
---
[](https://gitpod.io/from-referrer/)
|
t-data |
7/4 |
Mathlib/Data/Finsupp/Pointwise.lean |
1 |
6 |
['Paul-Lez', 'eric-wieser', 'github-actions'] |
nobody |
54-39914 1 month ago |
96-28212 3 months ago |
96-28261 96 days |
25070 |
erdOne author:erdOne |
feat(EllipticCurve): rational points on singular cuspidal cubics |
---
[](https://gitpod.io/from-referrer/)
|
t-algebraic-geometry |
123/0 |
Mathlib.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Singular/Cusp.lean |
2 |
9 |
['Multramate', 'acmepjz', 'erdOne', 'github-actions', 'kckennylau'] |
nobody |
54-30369 1 month ago |
60-6770 1 month ago |
60-6765 60 days |
25225 |
xcloudyunx author:xcloudyunx |
feat(Combinatorics/SimpleGraph): Eulerian walk in connected graph contains all vertices |
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-combinatorics
|
16/0 |
Mathlib/Combinatorics/SimpleGraph/Trails.lean |
1 |
3 |
['IvanRenison', 'github-actions'] |
nobody |
53-26052 1 month ago |
54-17464 1 month ago |
54-17518 54 days |
25153 |
eric-wieser author:eric-wieser |
feat(Algebra/ModEq): a lemma about `[PMOD (n • p)]` |
This ultimately didn't end up very useful to me, but I think it's still a nice result.
---
[](https://gitpod.io/from-referrer/)
|
t-number-theory |
20/0 |
Mathlib/Algebra/ModEq.lean |
1 |
3 |
['YaelDillies', 'eric-wieser', 'github-actions'] |
nobody |
52-77642 1 month ago |
56-43381 1 month ago |
56-43362 56 days |
24804 |
Moises-Herradon-Cueto author:Moises-Herradon-Cueto |
feat(CategoryTheory/Limits/Preserves/Shapes): show that if a functor preserves limits, so does `Over.post` |
If a functor `F` preserves limits (of a certain shape, finite, or of a certain size), then so does the induced functor on `Over` categories.
From Toric
Co-authored-by: Yaël Dillies
---
[](https://gitpod.io/from-referrer/)
|
toric
new-contributor
t-category-theory
|
125/0 |
Mathlib.lean,Mathlib/CategoryTheory/Limits/Preserves/Shapes/Over.lean,Mathlib/CategoryTheory/WithTerminal/Basic.lean |
3 |
17 |
['Moises-Herradon-Cueto', 'YaelDillies', 'erdOne', 'github-actions', 'joelriou'] |
nobody |
52-72320 1 month ago |
53-48262 1 month ago |
59-52655 59 days |
24412 |
pechersky author:pechersky |
feat(UniformSpace/Ultra/Constructions): IsUltraUniformity.{bot,top} |
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-topology
|
29/0 |
Mathlib/Order/Filter/Bases/Basic.lean,Mathlib/Topology/UniformSpace/Defs.lean,Mathlib/Topology/UniformSpace/Ultra/Basic.lean,Mathlib/Topology/UniformSpace/Ultra/Constructions.lean |
4 |
6 |
['github-actions', 'pechersky', 'urkud'] |
urkud assignee:urkud |
52-7033 1 month ago |
52-10243 1 month ago |
77-7200 77 days |
24095 |
lecopivo author:lecopivo |
feat: `fun_prop` for Is(Bounded)LinearMap + notation `fun x ↦L[R] f x` |
Sets up `fun_prop` for `IsLinearMap` and `IsBoundedLinearMap` also adds notation `fun x ↦ₗ[R] f x` and `fun x ↦L[R] f x` to write bundled versions like lambda function instead of the currently used pointfree notation. |
large-import
t-algebra
label:t-algebra$ |
352/22 |
Mathlib.lean,Mathlib/Algebra/Algebra/Bilinear.lean,Mathlib/Algebra/Module/LinearMap/Defs.lean,Mathlib/Algebra/Module/LinearMap/End.lean,Mathlib/Algebra/Module/LinearMap/Pi.lean,Mathlib/Algebra/Module/LinearMap/Prod.lean,Mathlib/Analysis/Normed/Operator/BoundedLinearMaps.lean,scripts/noshake.json |
8 |
22 |
['eric-wieser', 'github-actions', 'lecopivo'] |
nobody |
51-36431 1 month ago |
51-36431 1 month ago |
51-54813 51 days |
25322 |
thorimur author:thorimur |
style: use simplex notation (`⦋n⦌`) where possible |
`StandardSimplex.mk n` is replaced with `⦋n⦌` where possible (except in notation and macros, which are left untouched). This includes opening `Simplicial` in two files. Also, outdated and unused `local notation` `[n]` for `StandardSimplex.mk n` is removed.
---
[](https://gitpod.io/from-referrer/)
|
t-topology |
38/39 |
Mathlib/AlgebraicTopology/CechNerve.lean,Mathlib/AlgebraicTopology/MooreComplex.lean,Mathlib/AlgebraicTopology/SimplexCategory/Basic.lean,Mathlib/AlgebraicTopology/SimplicialObject/Basic.lean,Mathlib/AlgebraicTopology/SimplicialSet/Coskeletal.lean,Mathlib/AlgebraicTopology/SimplicialSet/NerveAdjunction.lean,Mathlib/AlgebraicTopology/SimplicialSet/StdSimplex.lean |
7 |
1 |
['github-actions'] |
nobody |
50-8881 1 month ago |
50-19460 1 month ago |
50-19510 50 days |
25343 |
plp127 author:plp127 |
docs(Topology/Perfect): Mention dense-in-itself |
The file `Mathlib/Topology/Perfect` defines a "nonstandard" predicate `Preperfect C` to mean that every point of `C` is an accumulation point of `C`. This property already has a name, it is called [dense-in-itself](https://en.wikipedia.org/wiki/Dense-in-itself). This PR adds this name to the docs.
---
[](https://gitpod.io/from-referrer/)
|
t-topology
documentation
|
7/7 |
Mathlib/Topology/Perfect.lean |
1 |
1 |
['github-actions'] |
nobody |
48-56657 1 month ago |
48-56735 1 month ago |
48-56717 48 days |
25337 |
alreadydone author:alreadydone |
feat(RingTheory): invertible modules and Picard group |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
535/0 |
Mathlib.lean,Mathlib/RingTheory/Finiteness/Cardinality.lean,Mathlib/RingTheory/PicardGroup.lean,docs/references.bib |
4 |
37 |
['alreadydone', 'erdOne', 'github-actions', 'kckennylau'] |
nobody |
48-5094 1 month ago |
49-14816 1 month ago |
49-14804 49 days |
25401 |
digama0 author:digama0 |
feat(Util): SuppressSorry option |
See also leanprover/lean4#8611 and [#lean4 > Silent sorry @ 💬](https://leanprover.zulipchat.com/#narrow/channel/270676-lean4/topic/Silent.20sorry/near/503537964). This is a stop-gap solution while leanprover/lean4#8611 is underway, but it works about as well as any other built in option. Hooking declaration elaborators turns out to be a very powerful technique.
---
[](https://gitpod.io/from-referrer/)
|
t-meta |
342/0 |
Mathlib.lean,Mathlib/Util/CommandElabHook.lean,Mathlib/Util/SuppressSorry.lean,MathlibTest/suppressSorry.lean |
4 |
13 |
['digama0', 'eric-wieser', 'github-actions'] |
nobody |
45-11087 1 month ago |
45-35421 1 month ago |
46-45768 46 days |
25453 |
JovanGerb author:JovanGerb |
perf(Algebra/Homology/HomotopyCategory): use explicit universe parameter in `Category` |
As we have seen before, writing `Category.{v}` instead of `Category` avoids a nasty universe level metavariable, and this helps to speed up unification. The changes in this PR are somewhat arbitrary, but it serves as an example for this principle.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
9/6 |
Mathlib/Algebra/Homology/HomotopyCategory/DegreewiseSplit.lean,Mathlib/Algebra/Homology/HomotopyCategory/MappingCone.lean,Mathlib/Algebra/Homology/HomotopyCategory/Triangulated.lean |
3 |
5 |
['JovanGerb', 'github-actions', 'leanprover-bot'] |
nobody |
44-62075 1 month ago |
45-29723 1 month ago |
45-29774 45 days |
25089 |
Bergschaf author:Bergschaf |
feat(Order/Sublocale): definition of sublocales |
There are several possible definition of sublocales. I used one from [nlab](https://ncatlab.org/nlab/show/sublocale) which states that a sublocale is a subset of a locale which is closed under all meets and for any ∈ S and x ∈ X, we have x ⇨ s ∈ S.
This PR also includes an order isomorphism between (Nucleus)ᵒᵈ and Sublocale.
---
I am open to better name suggestions for the order isomorphism.
- [x] depends on: #24941
[](https://gitpod.io/from-referrer/)
|
maintainer-merge
t-order
|
265/8 |
Mathlib.lean,Mathlib/Order/Hom/Lattice.lean,Mathlib/Order/Nucleus.lean,Mathlib/Order/Sublocale.lean,Mathlib/Order/Synonym.lean,docs/references.bib |
6 |
71 |
['Bergschaf', 'YaelDillies', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'xhalo32'] |
nobody |
42-30305 1 month ago |
42-30305 1 month ago |
56-9726 56 days |
25481 |
kbuzzard author:kbuzzard |
chore: refactor Algebra.TensorProduct.rightAlgebra |
The declaration `Algebra.TensorProduct.rightAlgebra` makes `A ⊗[R] B` into a `B`-algebra (here `R` is a `CommSemiring`, `A` is a `Semiring` and an `R`-algebra, and `B` is a `CommSemiring` and an `R`-algebra). It is not an instance because if A = B it causes a diamond. However in the many cases where A isn't B, it can occasionally be useful.
However one could imagine that in the many cases where an R-module `M` also isn't `B`, it might occasionally be useful to make `M ⊗[R] B` into a `B`-module (and indeed I am finding this in FLT). With the current definition of `Algebra.TensorProduct.rightAlgebra` this is difficult to do without causing diamonds in the case when `M` happens to be an `R`-algebra (by which I mean "I failed to do this in finite time").
One fix for this is just to redefine `Algebra.TensorProduct.rightAlgebra` so that the `smul` field is
```
smul b ab := TensorProduct.comm _ _ _ (b • (TensorProduct.comm _ _ _ ab))
```
i.e. literally "swap the product around, use mathlib's instance making `B ⊗[R] A` into a `B`-algebra, and then swap back". Then the same definition can be used to make `M ⊗[R] B` into a `B`-module and on the odd occasion where this point of view is useful, there is no diamond. This is what we do in this PR. After adding one simp lemma there is no breakage at all in mathlib. Furthermore, for those who have observed that we want to build on this algebra instance sometimes and, for example, add instances of the form "if M is finite over R then M ⊗[R] B is finite over B" -- these instances are really easy to add now with this new definition, because you simply pull back the analogous finite left module instance along the isomorphism M ⊗[R] B = B ⊗[R] M. Examples (from FLT, where the right action is put in a scope):
```
scoped instance [Module.Finite R M] : Module.Finite A (M ⊗[R] A) :=
Module.Finite.equiv (Module.TensorProduct.comm R A M)
scoped instance [Module.Free R M] : Module.Free A (M ⊗[R] A) :=
Module.Free.of_equiv (Module.TensorProduct.comm R A M)
```
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
33/6 |
Mathlib/RingTheory/TensorProduct/Basic.lean |
1 |
4 |
['github-actions', 'kbuzzard', 'leanprover-bot'] |
nobody |
41-73092 1 month ago |
44-52639 1 month ago |
44-52894 44 days |
25600 |
Komyyy author:Komyyy |
refactor: lemma expressing `ContinuousAt` using a punctured neighbourhood |
---
This lemma is used to prove that the Riemann zeta function is meromorphic in #25597.
[](https://gitpod.io/from-referrer/)
|
maintainer-merge
t-topology
|
4/0 |
Mathlib/Topology/ContinuousOn.lean |
1 |
5 |
['Komyyy', 'github-actions', 'grunweg'] |
nobody |
41-22178 1 month ago |
41-22178 1 month ago |
41-34063 41 days |
24850 |
pechersky author:pechersky |
feat(Topology/UniformSpace/Ultra): uniform spaces induced by pseudometrics are ultra if system is ultra |
Any uniform space has a natural system of pseudometrics definable on it,
comprised of those pseudometrics constructed from a descending chain of
equivalence relation entourages. In a nonarchimedean uniformity, this pseudometric system
induces the uniformity.
---
[](https://gitpod.io/from-referrer/)
- [x] depends on: #23111 |
t-topology |
509/1 |
Mathlib.lean,Mathlib/Topology/MetricSpace/BundledFun.lean,Mathlib/Topology/UniformSpace/Ultra/Pseudometrizable.lean |
3 |
8 |
['ADedecker', 'fpvandoorn', 'github-actions', 'mathlib4-dependent-issues-bot', 'pechersky'] |
nobody |
39-85346 1 month ago |
39-85409 1 month ago |
55-30944 55 days |
25730 |
xroblot author:xroblot |
feat(ZLattice/Covolume): add `covolume_div_covolume_eq_relindex` |
Add the following result:
Let `L₁` be a sub-`ℤ`-lattice of `L₂`. Then the index of `L₁` inside `L₂` is equal to `covolume L₁ / covolume L₂`.
---
- [x] depends on: #22940
- [x] depends on: #23759
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #22961.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/22961* |
t-algebra label:t-algebra$ |
66/3 |
Mathlib/Algebra/Module/ZLattice/Basic.lean,Mathlib/Algebra/Module/ZLattice/Covolume.lean,Mathlib/GroupTheory/Index.lean,Mathlib/LinearAlgebra/Determinant.lean |
4 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
37-78770 1 month ago |
37-79861 1 month ago |
37-79844 37 days |
25760 |
robin-carlier author:robin-carlier |
feat(CategoryTheory/Bicategory): (2,1)-categories and `Pith` |
This PR introduces a class `IsLocallyGroupoid` on bicategories, asserting that every hom-category has an `IsGroupoid` instance.
With this definition, `IsLocallyGroupoid (LocallyDiscrete C)` is correctly inferred.
Given a bicategory `B`, we introduce a type alias `Pith B` for `B` (realized as a one-field structure), and we equip it with a `Bicategory` instance where the hom-categories are the cores of the hom-categories of `B`. We show that this bicategory is a (2,1)-category, construct an inclusion pseudo-functor from `Pith B` to `B`, and show that every pseudofunctor from a (2,1)-category to `B` factors through this inclusion.
---
We can’t fully state the fact that `(pseudofunctorToPith F).comp (inclusion F)` "is" `F` because #18254 is still not merged.
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #25150.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/25150* |
t-category-theory |
191/0 |
Mathlib.lean,Mathlib/CategoryTheory/Bicategory/LocallyGroupoid.lean |
2 |
1 |
['github-actions'] |
nobody |
37-69796 1 month ago |
37-69869 1 month ago |
37-69852 37 days |
25736 |
robin-carlier author:robin-carlier |
feat(AlgebraicTopology/SimplexCategory/GeneratorsRelations/NormalForms): Normal forms for `P_σ`s |
We prove that admissible lists indeed provide a normal form for morphisms of satisfying `P_σ`.
To this end, we introduce `standardσ`, a construction that takes a list and turn it into a composition of `σ i`s in `SimplexCategoryGenRel`. We then prove that, thangs to the fifth simplicial identity, composition on the right corresponds to simplicial insertion in the list. This gives existence of a normal form for every morphism satisfying `P_σ`.
For unicity, we introduce an auxiliary function `simplicialEvalσ : (List ℕ) → ℕ → ℕ` and show that for admissible lists, it lifts to `ℕ` the `orderHom` attached to `toSimplexCategory.map standardσ`, and that we can recover elements of the list only by looking at values of this function.
Part of a series of PR formalising that `SimplexCategoryGenRel` is equivalent to `SimplexCategory`.
---
- [x] depends on: #21744
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #21745.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/21745* |
large-import
t-topology
t-category-theory
|
253/7 |
Mathlib/AlgebraicTopology/SimplexCategory/GeneratorsRelations/NormalForms.lean |
1 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
37-65369 1 month ago |
37-75059 1 month ago |
37-75045 37 days |
25795 |
dagurtomas author:dagurtomas |
chore(Condensed): introduce an abbrev for the equivalence of light condensed sets with a category of sheaves on a small site |
---
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #24522.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/24522* |
t-condensed |
39/0 |
Mathlib.lean,Mathlib/Condensed/Light/Small.lean |
2 |
1 |
['github-actions'] |
nobody |
37-63254 1 month ago |
37-63319 1 month ago |
37-63302 37 days |
25804 |
erdOne author:erdOne |
feat: `∑ z ∈ L, ‖z - x‖⁻ʳ` converges for lattices `L` |
---
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #21673.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/21673* |
t-analysis |
319/0 |
Mathlib.lean,Mathlib/Algebra/BigOperators/Group/Finset/Disjoint.lean,Mathlib/Algebra/Module/ZLattice/Summable.lean,Mathlib/Order/Disjointed.lean |
4 |
1 |
['github-actions'] |
nobody |
37-53830 1 month ago |
37-60529 1 month ago |
37-60512 37 days |
25788 |
Parcly-Taxel author:Parcly-Taxel |
feat: number of edges in the Turán graph |
We provide two theorems, the first `card_edgeFinset_turanGraph` providing the exact number of edges and the other `card_edgeFinset_turanGraph_le` providing a (slightly) looser bound whose main advantage is its lack of integer division/modulus operations.
The bound in `card_edgeFinset_turanGraph_le` is also the bound provided in [Motzkin and Straus (1965)](https://doi.org/10.4153%2FCJM-1965-053-6). |
large-import
t-combinatorics
|
132/0 |
Mathlib/Combinatorics/SimpleGraph/Turan.lean,Mathlib/Data/Nat/ModEq.lean |
2 |
2 |
['YaelDillies', 'github-actions'] |
nobody |
37-52332 1 month ago |
37-65285 1 month ago |
37-65270 37 days |
25724 |
bryangingechen author:bryangingechen |
chore: disable scheduled runs of stale issues workflow |
There's no point in having this run on schedule while it's still in limbo.
---
This also seems to have been [completely broken](https://github.com/leanprover-community/mathlib4/actions/workflows/stale.yml) since #21681, since the search string is too long. Maybe we should just delete this. |
CI |
1/2 |
.github/workflows/stale.yml |
1 |
1 |
['github-actions'] |
nobody |
37-50627 1 month ago |
38-1096 1 month ago |
38-1078 38 days |
25829 |
kbuzzard author:kbuzzard |
feat: add mulEquivHaarChar |
API for the positive real factor by which an continuous multiplicative equivalence scales a regular Haar measure on a locally compact topological group.
From FLT.
---
[](https://gitpod.io/from-referrer/)
|
t-measure-probability |
158/0 |
Mathlib.lean,Mathlib/MeasureTheory/Group/Measure.lean,Mathlib/MeasureTheory/Measure/Haar/MulEquivHaarChar.lean,Mathlib/MeasureTheory/Measure/Haar/Unique.lean |
4 |
1 |
['github-actions'] |
nobody |
37-17037 1 month ago |
37-18001 1 month ago |
37-18045 37 days |
25836 |
jt496 author:jt496 |
feat(SimpleGraph/FiveWheelLike): add the Andrásfai-Erdős-Sós theorem |
Add the Andrásfai-Erdős-Sós theorem `colorable_of_cliqueFree_lt_minDegree` which says that an `r + 1`-cliquefree graph `G` with sufficiently large minimum degree is `r`-colorable.
Co-authored-by: Lian Bremner Tattersall
---
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #25313.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/25313* |
large-import
t-combinatorics
|
307/4 |
Mathlib/Combinatorics/SimpleGraph/FiveWheelLike.lean |
1 |
1 |
['github-actions'] |
nobody |
36-66941 1 month ago |
36-67790 1 month ago |
36-67776 36 days |
25842 |
mitchell-horner author:mitchell-horner |
feat(Combinatorics/SimpleGraph): define turanDensity |
Define the Turán density `turanDensity H` of a simple graph `H`: `turanDensity H` is the limit of `extremalNumber n H / n.choose 2` as `n` approaches `∞`.
Also prove
- the Turán density of a simple graph is well-defined, that is, the limit `extremalNumber n H / n.choose 2` as `n` approaches `∞` exists,
- `extremalNumber n H` is asymptotically equivalent to `turanDensity H * n.choose 2` as `n` approaches `∞`.
---
- [x] depends on: #19865
- [x] depends on: #20681
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #20171.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/20171* |
t-combinatorics |
210/0 |
Mathlib.lean,Mathlib/Combinatorics/SimpleGraph/Extremal/Basic.lean,Mathlib/Combinatorics/SimpleGraph/Extremal/TuranDensity.lean,Mathlib/Combinatorics/SimpleGraph/Finite.lean,Mathlib/Data/Sym/Sym2.lean,Mathlib/Order/Monotone/Basic.lean |
6 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
b-mehta assignee:b-mehta |
36-47594 1 month ago |
36-47594 1 month ago |
36-52727 36 days |
25680 |
kim-em author:kim-em |
chore: remove some `Nat` shortcut instances |
This PR continues the work from #24928.
Original PR: https://github.com/leanprover-community/mathlib4/pull/24928 |
|
0/9 |
Mathlib/Algebra/Ring/Divisibility/Basic.lean,Mathlib/Data/List/TakeDrop.lean,Mathlib/Data/Nat/Basic.lean |
3 |
10 |
['b-mehta', 'eric-wieser', 'github-actions', 'leanprover-bot', 'mattrobball'] |
nobody |
36-46943 1 month ago |
39-16054 1 month ago |
39-16035 39 days |
25966 |
b-reinke author:b-reinke |
feat(GroupTheory/FreeGroup/ReducedWords): add theory of reduced words |
This PR continues the work from #23368.
Original PR: https://github.com/leanprover-community/mathlib4/pull/23368 |
t-algebra label:t-algebra$ |
104/0 |
Mathlib.lean,Mathlib/GroupTheory/FreeGroup/ReducedWords.lean |
2 |
2 |
['b-reinke', 'github-actions'] |
nobody |
33-45074 1 month ago |
33-45084 1 month ago |
33-45132 33 days |
25965 |
b-reinke author:b-reinke |
feat(Algebra/BigOperators/Finprod): add powerset projection lemmas |
This PR continues the work from #23926.
Original PR: https://github.com/leanprover-community/mathlib4/pull/23926 |
|
30/0 |
Mathlib/Algebra/BigOperators/Finprod.lean,Mathlib/Data/Set/Image.lean |
2 |
2 |
['b-reinke', 'github-actions'] |
joelriou assignee:joelriou |
33-40467 1 month ago |
33-45808 1 month ago |
33-45789 33 days |
25992 |
Multramate author:Multramate |
feat(RingTheory/Ideal/Span): add pair lemmas |
This PR continues the work from #25323.
Original PR: https://github.com/leanprover-community/mathlib4/pull/25323 |
|
131/31 |
Mathlib/Algebra/Module/PID.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Affine/Point.lean,Mathlib/RingTheory/DedekindDomain/AdicValuation.lean,Mathlib/RingTheory/Ideal/Maps.lean,Mathlib/RingTheory/Ideal/Span.lean |
5 |
2 |
['Multramate', 'github-actions'] |
nobody |
33-21111 1 month ago |
33-21186 1 month ago |
33-21167 33 days |
26009 |
linesthatinterlace author:linesthatinterlace |
feat: Add `Vector`/`List.Vector` equivalence |
This PR continues the work from #25050.
Original PR: https://github.com/leanprover-community/mathlib4/pull/25050 |
migrated-from-branch |
125/17 |
Mathlib/Data/Vector/Basic.lean,Mathlib/Data/Vector/Defs.lean,Mathlib/Logic/Equiv/Array.lean |
3 |
2 |
['github-actions', 'linesthatinterlace'] |
nobody |
32-66154 1 month ago |
32-66154 1 month ago |
32-68679 32 days |
25854 |
robin-carlier author:robin-carlier |
feat(CategoryTheory/Monoidal/Opposites): monoid objects internal to the monoidal opposite |
We construct an equivalence between monoid objects internal to a monoidal category `C`, and monoid objects internal to its monoidal opposite `Cᴹᵒᵖ`. This is done by adding `Mon_Class` and `IsMon_Hom` instance to the relevant objects, as well as by recording an explicit equivalence of categories `Mon_ C ≌ Mon_ Cᴹᵒᵖ`.
---
- [x] depends on: #25826
I made this depend on #25549 rather than making it work with the current def only to have it refactored when #25549 is merged.
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #25626.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/25626* |
t-category-theory |
112/0 |
Mathlib.lean,Mathlib/CategoryTheory/Monoidal/Opposite/Mon_.lean |
2 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
32-41348 1 month ago |
34-39291 1 month ago |
34-39274 34 days |
26054 |
FMLJohn author:FMLJohn |
feat(RingTheory/GradedAlgebra/Homogeneous/Subsemiring): homogeneous subsemirings of a graded semiring |
---
[](https://gitpod.io/from-referrer/)
In this pull request, we have defined homogeneous subsemirings of `GradedRing 𝒜` where `𝒜 : ι → σ`, `SetLike σ A` and `AddSubmonoidClass σ A`.
## Main definitions
For any `R : Subsemiring A`:
* `Subsemiring.IsHomogeneous 𝒜 R`: The property that a subsemiring is closed under `GradedRing.proj`.
* `HomogeneousSubsemiring 𝒜`: The structure extending subsemirings which satisfy `Subsemiring.IsHomogeneous`. |
t-algebra label:t-algebra$ |
120/0 |
Mathlib.lean,Mathlib/RingTheory/GradedAlgebra/Homogeneous/Subsemiring.lean |
2 |
1 |
['github-actions'] |
nobody |
32-34780 1 month ago |
32-35752 1 month ago |
32-35735 32 days |
26076 |
joelriou author:joelriou |
feat(AlgebraicTopology/SimplicialSet): uniqueness of the decomposition involving non-degenerate simplices |
Any simplex `x : X _⦋n⦌` of a simplicial set can be written in a unique way as `X.map f.op y` for an epimorphism `f : ⦋n⦌ ⟶ ⦋m⦌` and a non-degenerate `m`-simplex `y`.
---
This PR continues the work from #21103.
Original PR: https://github.com/leanprover-community/mathlib4/pull/21103 |
t-topology |
118/5 |
Mathlib/AlgebraicTopology/SimplexCategory/Basic.lean,Mathlib/AlgebraicTopology/SimplicialSet/Degenerate.lean |
2 |
2 |
['github-actions', 'joelriou'] |
nobody |
31-68286 1 month ago |
31-68297 1 month ago |
31-68343 31 days |
25183 |
YaelDillies author:YaelDillies |
feat: convolution product on linear maps from a coalgebra to an algebra |
Construct the ring structure on linear maps `C → A` where `C` is a coalgebra and `A` an algebra, where multiplication is given by
`(f * g)(x) = ∑ f x₍₁₎ * g x₍₂₎` in Sweedler notation or
```
|
μ
| | / \
f * g = f g
| | \ /
δ
|
```
diagrammatically, where `μ` stands for multiplication and `δ` for comultiplication.
[Zulip](https://leanprover.zulipchat.com/#narrow/channel/217875-Is-there-code-for-X.3F/topic/.60Mul.60.20instance.20on.20algebra.20homomorphisms.20from.20monoid.20algebra)
From Toric
Co-authored-by: Michał Mrugała
Co-authored-by: Yunzhou Xie
---
[](https://gitpod.io/from-referrer/)
|
toric
t-algebra
label:t-algebra$ |
137/0 |
Mathlib.lean,Mathlib/RingTheory/Coalgebra/Convolution.lean |
2 |
15 |
['YaelDillies', 'erdOne', 'eric-wieser', 'github-actions', 'smorel394'] |
nobody |
31-67282 1 month ago |
55-31843 1 month ago |
55-35764 55 days |
26099 |
grunweg author:grunweg |
feat: add IsEmbedding.sumElim_of_separatingNhds |
Characterise when the Sum.elim of two inducing maps resp. embeddings is an embedding,
and deduce that the ranges of the two maps lying in separated neighbourhoods suffices.
This is used in my bordism theory project.
Co-authored by: @plp127
---
This PR was manually re-created (and migrated to a fork at the same time) from #22137, since that seemed easiest.
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-topology
|
115/0 |
Mathlib/Data/Sum/Basic.lean,Mathlib/Topology/Constructions/SumProd.lean |
2 |
1 |
['github-actions'] |
nobody |
31-49186 1 month ago |
31-49246 1 month ago |
31-49237 31 days |
25858 |
themathqueen author:themathqueen |
feat(RingTheory/Coalgebra/MulOpposite): coalgebra instance for MulOpposite |
Adding an instance for `Aᵐᵒᵖ` being an `R`-coalgebra when `A` is.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-algebra
label:t-algebra$ |
112/0 |
Mathlib.lean,Mathlib/RingTheory/Coalgebra/MulOpposite.lean |
2 |
1 |
['github-actions'] |
nobody |
31-22953 1 month ago |
35-54752 1 month ago |
35-54796 35 days |
26154 |
ADedecker author:ADedecker |
refactor: add refactored APIs for algebraic filter bases |
This PR continues the work from #18437.
Original PR: https://github.com/leanprover-community/mathlib4/pull/18437 |
t-topology |
651/0 |
Mathlib.lean,Mathlib/Topology/Algebra/FilterBasis.lean,Mathlib/Topology/Algebra/FilterBasisNew.lean,Mathlib/Topology/Algebra/Nonarchimedean/Bases.lean,Mathlib/Topology/Algebra/Nonarchimedean/BasesNew.lean |
5 |
2 |
['ADedecker', 'github-actions'] |
nobody |
30-56263 1 month ago |
30-56263 1 month ago |
30-56321 30 days |
26157 |
erdOne author:erdOne |
chore(RingTheory): Merge `Mathlib/RingTheory/LocalRing/ResidueField/Algebraic.lean` into `Instances.lean` |
This was added a week ago by myself so I don't think a deprecation is needed
---
[](https://gitpod.io/from-referrer/)
|
file-removed |
22/34 |
Mathlib.lean,Mathlib/NumberTheory/RamificationInertia/Unramified.lean,Mathlib/RingTheory/LocalRing/ResidueField/Algebraic.lean,Mathlib/RingTheory/LocalRing/ResidueField/Instances.lean |
4 |
1 |
['github-actions'] |
nobody |
30-51865 1 month ago |
30-52026 1 month ago |
30-52078 30 days |
26159 |
upobir author:upobir |
feat(Algebra/QuadraticDiscriminant): Adding inequalities on quadratic from inequalities on discriminant |
This PR continues the work from #24517.
Original PR: https://github.com/leanprover-community/mathlib4/pull/24517 |
t-algebra label:t-algebra$ |
35/0 |
Mathlib/Algebra/QuadraticDiscriminant.lean |
1 |
3 |
['github-actions', 'upobir'] |
nobody |
30-50571 1 month ago |
30-51007 1 month ago |
30-51050 30 days |
26156 |
oliver-butterley author:oliver-butterley |
feat(MeasureTheory.VectorMeasure) : add a definition of total variation for VectorMeasure |
This PR adds variation for any `VectorMeasure` using a supremum definition. Currently mathlib has `TotalVariation` defined for a signed measure using the Hahn-Jordan decomposition, but this doesn't generalise.
Motivation: generally this is an important concept but specifically as a step for proving RMK in the complex case which in turn is a step to prove the spectral theorem.
Co-authored-by: @yoh-tanimoto
This PR was migrated from #25442. PR divided into smaller pieces, this is just the definition without additional lemmas. PRs adding further results related to variation are:
* #26160
* #26165
* #26168 (shows that for `SignedMeasures` the two definitions of variation coincide)
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-measure-probability
|
354/0 |
Mathlib.lean,Mathlib/MeasureTheory/VectorMeasure/Variation/Defs.lean |
2 |
1 |
['github-actions'] |
nobody |
29-72333 29 days ago |
30-53350 1 month ago |
30-53398 30 days |
26200 |
adomani author:adomani |
fix: add label when landrun fails |
Adds the `permission-denied` label on PRs that get blocked by landrun.
---
[](https://gitpod.io/from-referrer/)
|
CI |
68/8 |
.github/build.in.yml,.github/workflows/bors.yml,.github/workflows/build.yml,.github/workflows/build_fork.yml |
4 |
1 |
['github-actions'] |
nobody |
29-67827 29 days ago |
29-67833 29 days ago |
29-67878 29 days |
26225 |
Raph-DG author:Raph-DG |
feat(AlgebraicGeometry): Add some minimal API for orders on schemes |
In this PR we add some minimal api for the ordering on schemes defined in #26204. We chose split these PRs because we expect there will be more discussion about this API, and having the preorder instance is useful in its own right without much added API.
- [] depends on: #26204
---
[](https://gitpod.io/from-referrer/)
|
t-algebraic-geometry |
16/0 |
Mathlib/AlgebraicGeometry/Properties.lean,Mathlib/AlgebraicGeometry/Scheme.lean |
2 |
1 |
['github-actions'] |
nobody |
29-47241 29 days ago |
29-47250 29 days ago |
29-47294 29 days |
26130 |
kmill author:kmill |
feat: make `reassoc_of%` be able to defer `Category` instance |
This PR modifies the elaboration of `reassoc_of%` so that the `Category` instance can be synthesized later, like any other instance metavariable, rather than needing to be synthesized up front, when the category itself might not yet be known.
This fixes an issue reported by Robert Maxton [on Zulip](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/reassoc_of.25.20misleading.20error/near/524678383), where in the following `reassoc_of% Sigma.ι_desc` was failing.
```lean
import Mathlib.CategoryTheory.Limits.Shapes.Products
open CategoryTheory Limits
set_option autoImplicit true
variable {C : Type u} [Category.{v, u} C]
{β : Type w} {f : β → C} [HasCoproduct f] {P : C}
(p : (b : β) → f b ⟶ P) (b : β)
example {Q : C} (g : P ⟶ Q) : Sigma.ι f b ≫ Sigma.desc p ≫ g = p b ≫ g := by
rw [reassoc_of% Sigma.ι_desc]
```
Without this PR, a workaround is writing `reassoc_of% @Sigma.ι_desc`.
The PR adds `Lean.Meta.withEnsuringLocalInstance` for temporarily adding a metavariable as a local instance if it can't yet be synthesized.
---
[](https://gitpod.io/from-referrer/)
|
t-meta |
91/20 |
Mathlib/Lean/Meta/Basic.lean,Mathlib/Tactic/CategoryTheory/IsoReassoc.lean,Mathlib/Tactic/CategoryTheory/Reassoc.lean,MathlibTest/CategoryTheory/Reassoc.lean |
4 |
6 |
['github-actions', 'kmill', 'leanprover-bot', 'sgouezel'] |
nobody |
29-26485 29 days ago |
30-83776 1 month ago |
30-83758 30 days |
25883 |
pfaffelh author:pfaffelh |
feat: introduce Gram matrices |
A Gram matrix has entry `⟪v i, v j⟫` at `i j : n`, where `v : n → α` is an `InnerProductSpace 𝕜 α`.
Give this notion and show that Gram matrices are positive semi-definite.
This will be used later in order to show that the covariance matrix for Brownian Motion is positive semi-definite.
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #24575.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/24575* |
migrated-from-branch
new-contributor
|
157/2 |
Mathlib.lean,Mathlib/Analysis/InnerProductSpace/GramMatrix.lean,Mathlib/MeasureTheory/Function/L2Space.lean |
3 |
8 |
['eric-wieser', 'github-actions', 'pfaffelh'] |
nobody |
29-22590 29 days ago |
35-23840 1 month ago |
35-24192 35 days |
26240 |
grunweg author:grunweg |
perf(CommandLinterLinter): use Substring more |
Probably, these changes make little difference, but let's find out.
---
[](https://gitpod.io/from-referrer/)
|
t-linter
RFC
|
14/15 |
Mathlib/Tactic/Linter/CommandStart.lean |
1 |
5 |
['github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot'] |
nobody |
29-20641 29 days ago |
29-20641 29 days ago |
29-25253 29 days |
26258 |
kckennylau author:kckennylau |
feat(Topology): induction for sheafification |
---
I currently have binary and unary operation, which should be enough for sheaves.
[](https://gitpod.io/from-referrer/)
|
t-topology |
62/1 |
Mathlib/Topology/Sheaves/LocalPredicate.lean |
1 |
1 |
['github-actions'] |
nobody |
28-34271 28 days ago |
28-34380 28 days ago |
28-34442 28 days |
26061 |
kckennylau author:kckennylau |
feat(AlgebraicGeometry): define Projective Space |
This defines the projective space over a scheme, indexed by an arbitrary type.
---
Zulip discussion: [#maths > Projective Space](https://leanprover.zulipchat.com/#narrow/channel/116395-maths/topic/Projective.20Space/with/524057860)
[](https://gitpod.io/from-referrer/)
|
t-algebraic-geometry |
63/0 |
Mathlib.lean,Mathlib/AlgebraicGeometry/ProjectiveSpace.lean |
2 |
14 |
['callesonne', 'erdOne', 'github-actions', 'kckennylau'] |
nobody |
28-32146 28 days ago |
32-13410 1 month ago |
32-13456 32 days |
26259 |
Raph-DG author:Raph-DG |
feat(Topology): Connecting different notions of locally finite |
In this PR we connect the notions of local finiteness of an indexed family of sets (as in LocallyFinite) and of a set of sets (as in Function.locallyFinsuppWithin)
---
[](https://gitpod.io/from-referrer/)
|
t-topology |
32/0 |
Mathlib/Topology/LocallyFinsupp.lean |
1 |
3 |
['Raph-DG', 'github-actions', 'kckennylau'] |
nobody |
27-72014 27 days ago |
28-34175 28 days ago |
28-34217 28 days |
26120 |
vasnesterov author:vasnesterov |
feat(Data/Seq): `modify` and `set` operations for `Seq` |
Introduce `modify` and `set` operations for sequences, along with a few lemmas about them.
---
- [x] depends on: #20071
[](https://gitpod.io/from-referrer/)
This PR continues the work from #20160.
Original PR: https://github.com/leanprover-community/mathlib4/pull/20160 |
t-data |
69/0 |
Mathlib/Data/Seq/Seq.lean |
1 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'vasnesterov'] |
nobody |
27-49259 27 days ago |
31-30595 1 month ago |
31-30645 31 days |
25837 |
jt496 author:jt496 |
feat(Combinatorics/SimpleGraph): add homOfConnectedComponents and related results |
Given homomorphisms of each connected component of `G : SimpleGraph α` into `H : SimpleGraph β `give the corresponding `G →g H`
Hence prove that G is n - colorable iff each connected component is n - colorable.
Also prove that G is 2-colorable iff it does not contain an odd length loop (closed walk).
I wasn't sure where to put this - it probably belongs in SimpleGraph.ConcreteColorings?
---
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #24546.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/24546* |
t-combinatorics |
36/0 |
Mathlib/Combinatorics/SimpleGraph/Coloring.lean,Mathlib/Combinatorics/SimpleGraph/ConcreteColorings.lean,Mathlib/Combinatorics/SimpleGraph/Connectivity/Connected.lean |
3 |
1 |
['github-actions'] |
nobody |
27-45539 27 days ago |
36-67673 1 month ago |
36-67657 36 days |
26284 |
plp127 author:plp127 |
feat: faster implementation of `Nat.primeFactorsList` + `@[csimp]` lemma |
Add a function `Nat.primeFactorsListFast` that `#eval`s faster, and a `@[csimp]` lemma `Nat.primeFactorsList_eq_primeFactorsListFast` that shows `Nat.primeFactorsList = Nat.primeFactorsListFast`.
---
[](https://gitpod.io/from-referrer/)
|
t-data |
95/0 |
Mathlib/Data/Nat/Factors.lean |
1 |
1 |
['github-actions'] |
nobody |
26-85243 26 days ago |
26-85266 26 days ago |
27-12782 27 days |
26301 |
Ivan-Sergeyev author:Ivan-Sergeyev |
feat(LinearAlgebra/Matrix/Determinant/TotallyUnimodular): |
Empty matrices are totally unimodular.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-algebra
label:t-algebra$ |
15/0 |
Mathlib/LinearAlgebra/Matrix/Determinant/TotallyUnimodular.lean |
1 |
1 |
['github-actions'] |
nobody |
26-52633 26 days ago |
26-52643 26 days ago |
26-52687 26 days |
26189 |
tb65536 author:tb65536 |
feat(FieldTheory/Galois/Basic): Add simp-lemma for `FixedPoints.intermediateField` |
This PR adds a simp-lemma `FixedPoints.mem_intermediateField_iff` for the definition `FixedPoints.intermediateField`.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
4/0 |
Mathlib/FieldTheory/Galois/Basic.lean |
1 |
1 |
['github-actions'] |
nobody |
26-46143 26 days ago |
26-46143 26 days ago |
30-17393 30 days |
26308 |
LessnessRandomness author:LessnessRandomness |
feat(Analysis.NormedSpace): add normalized vectors |
---
Add normalized vectors to Mathlib (zero vector for zero vector, the corresponding unit vectors for nonzero vectors) |
new-contributor
t-analysis
|
65/0 |
Mathlib.lean,Mathlib/Analysis/NormedSpace/Normalized.lean |
2 |
1 |
['github-actions'] |
nobody |
26-44738 26 days ago |
26-44750 26 days ago |
26-44795 26 days |
25997 |
tb65536 author:tb65536 |
refactor(FieldTheory/Galois): Switch from `Fintype` to `Finite` |
This PR switches mathlib's Galois theory from `Fintype` to `Finite` to match the group theory library.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
59/61 |
Mathlib/FieldTheory/Galois/Basic.lean,Mathlib/FieldTheory/Galois/IsGaloisGroup.lean,Mathlib/FieldTheory/IntermediateField/Adjoin/Basic.lean,Mathlib/FieldTheory/KrullTopology.lean,Mathlib/FieldTheory/KummerExtension.lean,Mathlib/FieldTheory/PolynomialGaloisGroup.lean,Mathlib/NumberTheory/NumberField/CMField.lean,Mathlib/NumberTheory/NumberField/InfinitePlace/Ramification.lean |
8 |
1 |
['github-actions'] |
nobody |
26-44006 26 days ago |
26-44006 26 days ago |
32-50447 32 days |
26190 |
tb65536 author:tb65536 |
feat(FieldTheory/Galois/IsGaloisGroup): Subgroups of a Galois group are Galois groups |
This PR gives an instance `IsGaloisGroup H (FixedPoints.intermediateField H : IntermediateField K L) L` from `IsGaloisGroup G K L`, and a numerical corollary.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
11/0 |
Mathlib/FieldTheory/Galois/IsGaloisGroup.lean |
1 |
1 |
['github-actions'] |
nobody |
26-43103 26 days ago |
26-43104 26 days ago |
30-12705 30 days |
26319 |
Vierkantor author:Vierkantor |
ci: specify leanprover-community/mathlib4 when checking out master |
This PR makes it explicit that we want to run CI against the `master` branch from `leanprover-community/mathlib4` instead of another repo.
The new mathlib4-nightly-testing repo should run CI on the nightly branches as if they are already part of the `master` branch. But when checking them out, it defaults to looking for the branch in `leanprover-community/mathlib4-nightly-testing`, which does not exist. So a simple fix is to make the upstream repo name explicit.
A potential disadvantage: it will be harder to test CI changes by opening a pull request against one's own fork. (Which is what I did to test a few CI changes before).
---
This change makes sense to me but maybe there is a better option? I don't think we want to have custom CI in the other repo, because it will get obliterated next time we do an update.
[](https://gitpod.io/from-referrer/)
|
CI |
4/0 |
.github/build.in.yml,.github/workflows/bors.yml,.github/workflows/build.yml,.github/workflows/build_fork.yml |
4 |
1 |
['github-actions'] |
nobody |
26-37998 26 days ago |
26-38067 26 days ago |
26-38050 26 days |
26078 |
kckennylau author:kckennylau |
feat(AlgebraicGeometry): add x, y, px, py for points on elliptic curves |
---
Split from #25218.
[](https://gitpod.io/from-referrer/)
|
t-algebraic-geometry |
44/0 |
Mathlib/AlgebraicGeometry/EllipticCurve/Affine/Point.lean |
1 |
10 |
['MichaelStollBayreuth', 'Multramate', 'acmepjz', 'github-actions', 'kckennylau'] |
nobody |
26-19537 26 days ago |
31-58043 1 month ago |
31-58087 31 days |
26332 |
Timeroot author:Timeroot |
feat (ModelTheory/Definability): TermDefinable functions |
This PR continues the work from #23506.
Original PR: https://github.com/leanprover-community/mathlib4/pull/23506 |
large-import |
159/0 |
Mathlib/Data/Rel.lean,Mathlib/ModelTheory/Definability.lean,scripts/noshake.json |
3 |
2 |
['Timeroot', 'github-actions'] |
nobody |
26-4288 26 days ago |
26-4295 26 days ago |
26-4338 26 days |
23460 |
Timeroot author:Timeroot |
feat: Definition of `Clone` |
Basics about Clones. Part of #20051
---
- [x] depends on: #23459
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
326/0 |
Mathlib.lean,Mathlib/Algebra/Clone/Basic.lean,Mathlib/Algebra/Clone/Defs.lean,Mathlib/Data/Fin/Basic.lean |
4 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
26-3737 26 days ago |
26-3739 26 days ago |
26-5030 26 days |
26274 |
EtienneC30 author:EtienneC30 |
feat: api for symmetric bilinear forms |
Change the definition of `BilinForm.IsSymm` to make it a structure, in order to extend it to define `ContinuousBilinForm.IsPosSemidef` in #26315.
Prove polarization identity.
Prove two lemmas about `BilinForm.toMatrix`.
---
From Brownian motion
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
88/17 |
Mathlib/LinearAlgebra/BilinearForm/Orthogonal.lean,Mathlib/LinearAlgebra/BilinearForm/Properties.lean,Mathlib/LinearAlgebra/Matrix/BilinearForm.lean,Mathlib/RingTheory/Trace/Defs.lean |
4 |
2 |
['bryangingechen', 'github-actions'] |
nobody |
25-75918 25 days ago |
25-75918 25 days ago |
26-3890 26 days |
26255 |
vasnesterov author:vasnesterov |
feat(Analysis): radius of convergence for `FormalMultilinearSeries.compContinuousLinearMap` |
- Add basic lemmas `compContinuousLinearMap_id` and `compContinuousLinearMap_comp`.
- Prove lower and upper bounds for the convergence radius of `f.compContinuousLinearMap`.
- Prove `radius_compNeg`: the convergence radii of `f(x)` and `f(-x)` are equal.
---
In this PR I had to add `set_option linter.style.longFile 1700` in `Analytic/Basic.lean`.
I split this file in the next PR: #26270.
[](https://gitpod.io/from-referrer/)
This PR continues the work from #22531.
Original PR: https://github.com/leanprover-community/mathlib4/pull/22531 |
t-analysis |
148/11 |
Mathlib/Analysis/Analytic/Basic.lean,Mathlib/Analysis/Analytic/CPolynomial.lean,Mathlib/Analysis/Analytic/Constructions.lean,Mathlib/Analysis/Calculus/FormalMultilinearSeries.lean,Mathlib/Analysis/NormedSpace/OperatorNorm/NormedSpace.lean |
5 |
11 |
['github-actions', 'grunweg', 'vasnesterov'] |
grunweg assignee:grunweg |
25-32898 25 days ago |
26-49527 26 days ago |
28-22526 28 days |
25974 |
scholzhannah author:scholzhannah |
feat(Topology/Compactness/CompactlyCoherentSpace): compact coherentification (k-ification) |
This PR defines the notion of turning an arbitrary topological space into a compactly coherent space. Compactly coherent spaces are commonly referred to as "compactly generated spaces" or "k-spaces" in the literature while the operation of turning a space into such as space is called the "k-ification". There are however three different notions that are described with this name. To disambiguate we use the names "compactly coherent space" and "compactcoherentification" here. See [this wikipedia page](https://en.wikipedia.org/wiki/Compactly_generated_space) for an explanation of these notions.
This PR continues the work from #25318.
Original PR: https://github.com/leanprover-community/mathlib4/pull/25318
Co-authored-by: Floris van Doorn |
large-import
t-topology
|
175/5 |
Mathlib/Topology/Compactness/CompactlyCoherentSpace.lean |
1 |
2 |
['github-actions', 'scholzhannah'] |
nobody |
24-64434 24 days ago |
33-29954 1 month ago |
33-30002 33 days |
26428 |
Ruben-VandeVelde author:Ruben-VandeVelde |
feat: norm_num support for Int.fract |
---
[](https://gitpod.io/from-referrer/)
|
t-data |
44/0 |
Mathlib/Data/Rat/Floor.lean,MathlibTest/norm_num_ext.lean |
2 |
5 |
['Rob23oba', 'github-actions'] |
nobody |
23-24498 23 days ago |
23-24539 23 days ago |
23-69298 23 days |
26396 |
xroblot author:xroblot |
feat(RingTheory): define the dual of a basis for the trace and prove basic properties |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
133/28 |
Mathlib/LinearAlgebra/BilinearForm/Properties.lean,Mathlib/RingTheory/DedekindDomain/Different.lean,Mathlib/RingTheory/Trace/Basic.lean |
3 |
1 |
['github-actions'] |
nobody |
22-57743 22 days ago |
24-72448 24 days ago |
24-72498 24 days |
26453 |
jburroni author:jburroni |
feat(Data/PNat/Basic): add order-related instances to PNat |
Add `SuccAddOrder ℕ+` and `NoMaxOrder ℕ+` instances.
This allows, for example, the use of lemmas related to `Intervals` built with ℕ+.
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-data
new-contributor
|
18/0 |
Mathlib/Data/PNat/Basic.lean |
1 |
3 |
['eric-wieser', 'github-actions', 'jburroni'] |
nobody |
22-50782 22 days ago |
23-34640 23 days ago |
23-34685 23 days |
26358 |
plp127 author:plp127 |
feat(Topology): R1 spaces are quasisober |
This PR continues the work from #24054.
Original PR: https://github.com/leanprover-community/mathlib4/pull/24054 |
bench-after-CI
t-topology
|
23/9 |
Mathlib/Topology/Separation/Hausdorff.lean,Mathlib/Topology/Sober.lean |
2 |
16 |
['faenuccio', 'github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'plp127'] |
nobody |
22-26496 22 days ago |
22-26552 22 days ago |
25-51526 25 days |
26023 |
Garmelon author:Garmelon |
chore: add githelper.py script |
As described in the readme file, this somewhat opinionated script aims to help fix weird git repo setups and restore them to a standardized state that closely matches what `gh repo clone` does. Like `migrate_to_fork.py`, this script requires the user to have `git` and `gh` installed.
To use the script, run `scripts/githelper.py fix` in a git repo that is either a clone of mathlib or of a mathlib fork. The script will prompt you before making any changes, so the user retains control over the entire process. The script also prints the commands used.
`fix` is a subcommand so other git and github management tasks can be added in the future. Possible examples: Deleting branches of closed PRs, keeping the fork in sync with upstream, removing branches from a fork that was accidentally cloned with all mathlib branches included.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor |
490/0 |
scripts/README.md,scripts/githelper.py |
2 |
8 |
['Garmelon', 'bryangingechen', 'github-actions', 'jcommelin'] |
bryangingechen assignee:bryangingechen |
22-11425 22 days ago |
22-11425 22 days ago |
24-20700 24 days |
26287 |
mbkybky author:mbkybky |
feat(Data/ENat/Lattice): coercion to `WithBot ℕ∞` commutes with `biSup` |
The coercion from `ℕ∞` to `WithBot ℕ∞` commutes with `biSup` and `biInf`.
---
[](https://gitpod.io/from-referrer/)
|
t-data |
19/0 |
Mathlib/Data/ENat/Lattice.lean |
1 |
1 |
['github-actions'] |
nobody |
21-41253 21 days ago |
26-85193 26 days ago |
27-6543 27 days |
26462 |
PSchwahn author:PSchwahn |
feat(LinearAlgebra/Projection): add results about inverse of `Submodule.prodEquivOfIsCompl` |
Add two theorems `Submodule.prodEquivOfIsCompl_symm_apply` and `Submodule.prodEquivOfIsCompl_symm_add`, which are API for `Submodule.prodEquivOfIsCompl`.
We believe these theorems are useful; for example, we have used their statements in a [classification formalization project](https://github.com/LieLean/LowDimSolvClassification).
I am not sure whether the `prodEquivOfIsCompl_symm_apply` theorem should be tagged with `@[simp]`; this might lead to confluence issues. Opinions are welcome!
Co-authored by:
- [Viviana del Barco](https://github.com/vdelbarc)
- [Gustavo Infanti](https://github.com/GuQOliveira)
- [Exequiel Rivas](https://github.com/erivas)
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-algebra
label:t-algebra$ |
9/0 |
Mathlib/LinearAlgebra/Projection.lean |
1 |
5 |
['PSchwahn', 'github-actions', 'kckennylau'] |
nobody |
21-17992 21 days ago |
23-3626 23 days ago |
23-3751 23 days |
26489 |
chrisflav author:chrisflav |
refactor(RingTheory/RingHom): factor out proofs for `Algebra.FinitePresentation` |
The current way to use locality of a given property of algebras is to convert everything into the language of `RingHom`s and then for example the `RingHom.OfLocalizationSpanTarget` API. This has two disadvantages:
1. The ring hom property API fixes the universes of source and target to be the same, hence we unnecessarily lose out on some universe generality.
2. The results for `RingHom`s are proven by translating everything in terms of `Algebra`, so we duplicate the translation steps.
This PR refactors `RingHom.FinitePresentation` to do all locality proofs in the language of `Algebra`s and translate it into the corresponding `RingHom.OfLocalizationSpan{Target}` in the last step. We also streamline some of the translation proofs by unifying the API.
---
- [x] depends on: #22931
[](https://gitpod.io/from-referrer/)
This PR continues the work from #22930.
Original PR: https://github.com/leanprover-community/mathlib4/pull/22930 |
t-algebra label:t-algebra$ |
62/77 |
Mathlib/RingTheory/RingHom/FinitePresentation.lean |
1 |
4 |
['chrisflav', 'erdOne', 'github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
20-83301 20 days ago |
21-52454 21 days ago |
21-52501 21 days |
22662 |
plp127 author:plp127 |
feat: Localization.Away.lift (computably) |
This PR adds `Localization.Away.lift'` and `Localization.Away.lift`, computable alternatives to `Localization.awayLift`.
---
- [x] depends on: #24791
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
74/0 |
Mathlib/RingTheory/Localization/Away/Basic.lean |
1 |
12 |
['eric-wieser', 'github-actions', 'mathlib4-dependent-issues-bot', 'plp127', 'vihdzp'] |
nobody |
20-80392 20 days ago |
69-16075 2 months ago |
135-16058 135 days |
26510 |
alreadydone author:alreadydone |
feat(Matroid): exchange lemmas involving closure |
---
for #24350
[](https://gitpod.io/from-referrer/)
|
t-data
t-combinatorics
|
37/0 |
Mathlib/Data/Matroid/Closure.lean |
1 |
1 |
['github-actions'] |
nobody |
20-50058 20 days ago |
20-50084 20 days ago |
20-50129 20 days |
26155 |
xroblot author:xroblot |
feat(DedekindDomain/Different): add the transitivity formula |
This PR proves the transitivity formula for the different ideal.
It introduces ~~two~~ one increase~~s~~ in imports:
- `RingTheory.FractionalIdeal.Extended`: this is a short leaf file and I think the import makes sense there
- ~~`RingTheory.Localization.Defs.lean `: the file `Algebra.Algebra.Basic` is added since it is necessary to have the definition of `noZeroSMulDivisors` to get that some algebra map is injective. The import could be removed by stating the hypothesis as `Function.Injective (algebraMap * *)` but it is not the usual spelling (and cannot be synthesized by Lean). In the end, it appears that the increased import only affects three files so maybe it's fine.~~
The PR also adds two new instances:
- `FiniteDimensional (FractionRing A) (FractionRing B)` deduced from `Module.Finite A B` when `B` is a Dedekind domain.
- `IsScalarTower (FractionRing A) (FractionRing B) (FractionRing C)` deduced from `IsScalarTower A B C`
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebra
label:t-algebra$ |
207/4 |
Mathlib/RingTheory/DedekindDomain/Different.lean,Mathlib/RingTheory/DedekindDomain/IntegralClosure.lean,Mathlib/RingTheory/FractionalIdeal/Extended.lean,Mathlib/RingTheory/Localization/Basic.lean,Mathlib/RingTheory/Localization/FractionRing.lean |
5 |
13 |
['erdOne', 'github-actions', 'xroblot'] |
nobody |
19-54690 19 days ago |
22-55453 22 days ago |
27-52460 27 days |
25832 |
xroblot author:xroblot |
feat(FieldTheory/LinearDisjoint): `trace` (resp. `norm`) and `algebraMap` commutes |
For `A` and `B` two linearly disjoint `R`-subalgebras in a commutative algebra `S` and `b` a `R`-basis of `B`, we construct a `A`-basis of `S = A ⊔ B` from `b` (and a similar construction using a `R`-basis of `A`). Then, we prove in this situation that `trace` commutes with `algebraMap`, that is:
```lean
Algebra.trace A S (algebraMap B S x) = algebraMap R A (Algebra.trace R B x)
```
and a similar result for the norm.
We also add a similar basis construction for `A` and `B` two linearly disjoint intermediate fields with the hypothesis that `A.toSubalgebra ⊔ B.toSubalgebra = ⊤`. This hypothesis is equivalent to `A ⊔ B = ⊤` in many cases (for example, one of the two extensions is algebraic over the base field) but not always.
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebra
label:t-algebra$ |
161/9 |
Mathlib/FieldTheory/LinearDisjoint.lean,Mathlib/RingTheory/LinearDisjoint.lean |
2 |
23 |
['acmepjz', 'github-actions', 'xroblot'] |
nobody |
19-54386 19 days ago |
28-73966 28 days ago |
36-18951 36 days |
26357 |
javra author:javra |
feat(CategoryTheory): linear categories as `ModuleCat R`-enriched categories |
Continues #23826.
---
[](https://gitpod.io/from-referrer/)
|
large-import |
195/0 |
Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Monoidal/Basic.lean,Mathlib/CategoryTheory/Enriched/Linear.lean,Mathlib/CategoryTheory/Linear/Basic.lean,Mathlib/CategoryTheory/Monoidal/Linear.lean |
5 |
1 |
['github-actions'] |
nobody |
19-49867 19 days ago |
25-53251 25 days ago |
25-53302 25 days |
26351 |
RemyDegenne author:RemyDegenne |
feat: covering and packing numbers of sets in a metric space |
We define covering numbers of sets in a pseudo-metric space, which are minimal cardinalities of
`ε`-covers of sets. We also define the packing number, which is the maximal cardinality of
an `ε`-separated set.
From the Brownian motion project.
---
[](https://gitpod.io/from-referrer/)
|
t-topology |
261/0 |
Mathlib.lean,Mathlib/Topology/MetricSpace/CoveringNumbers.lean |
2 |
4 |
['ADedecker', 'YaelDillies', 'github-actions'] |
nobody |
19-49350 19 days ago |
25-66976 25 days ago |
25-67022 25 days |
26277 |
AntoineChambert-Loir author:AntoineChambert-Loir |
feat(RingTheory/Congruence/Hom): prove basic isomorphisms theorems for ring congruences |
This file contains elementary definitions involving congruence
relations and morphisms for semirings, rings, and algebras.
* `RingCon.ker`: the kernel of a monoid homomorphism as a congruence relation
* `RingCon.lift`, `RingCon.liftₐ`: the homomorphism / the algebra morphism
on the quotient given that the congruence is in the kernel
* `RingCon.map`, `RingCon.mapₐ`: homomorphism / algebra morphism
from a smaller to a larger quotient
* `RingCon.quotientKerEquivRangeS`, `RingCon.quotientKerEquivRange`,
`RingCon.quotientKerEquivRangeₐ` :
the first isomorphism theorem for semirings (using `RingHom.rangeS`),
rings (using `RingHom.range`) and algebras (using `AlgHom.range`).
* `RingCon.comapQuotientEquivRangeS`, `RingCon.comapQuotientEquivRange`,
`RingCon.comapQuotientEquivRangeₐ` : the second isomorphism theorem
for semirings (using `RingHom.rangeS`), rings (using `RingHom.range`)
and algebras (using `AlgHom.range`).
* `RingCon.quotientQuotientEquivQuotient`, `RingCon.quotientQuotientEquivQuotientₐ` :
the third isomorphism theorem for semirings (or rings) and algebras
It is an adaptation of what existed for multiplicative congruences (docs#Con) and is only useful for semirings which are not rings.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
555/2 |
Mathlib.lean,Mathlib/Algebra/Ring/Subsemiring/Basic.lean,Mathlib/Algebra/RingQuot.lean,Mathlib/RingTheory/Congruence/Basic.lean,Mathlib/RingTheory/Congruence/Defs.lean,Mathlib/RingTheory/Congruence/Hom.lean |
6 |
1 |
['github-actions'] |
nobody |
19-44225 19 days ago |
27-23312 27 days ago |
27-23360 27 days |
26543 |
vihdzp author:vihdzp |
feat(SetTheory/ZFC/VonNeumann): von Neumann hierarchy of sets |
Ported from #17027. For extra discussion on this PR, see [Zulip](https://leanprover.zulipchat.com/#narrow/channel/144837-PR-reviews/topic/.2317027.20.2C.20.2326518.20von.20Neumann.20hierarchy/with/526389347).
---
[](https://gitpod.io/from-referrer/)
|
t-set-theory
maintainer-merge
|
133/0 |
Mathlib.lean,Mathlib/SetTheory/Ordinal/Basic.lean,Mathlib/SetTheory/ZFC/Basic.lean,Mathlib/SetTheory/ZFC/VonNeumann.lean |
4 |
55 |
['alreadydone', 'github-actions', 'kckennylau', 'vihdzp'] |
nobody |
19-23880 19 days ago |
19-24121 19 days ago |
19-53659 19 days |
25947 |
qawbecrdtey author:qawbecrdtey |
feat(Data/Nat/Factors): added lemmas including `primeFactorsList_length_ne_zero` |
---
Added lemmas `primeFactorsList_length_ne_zero`, `primeFactorsList_prime_iff`, and `primeFactorsList_length_eq_one`.
```lean
theorem primeFactorsList_length_ne_zero (n : ℕ) : n.primeFactorsList.length ≠ 0 ↔ 2 ≤ n
theorem primeFactorsList_prime_iff {p : ℕ} : p.primeFactorsList = [p] ↔ p.Prime
@[simp]
theorem primeFactorsList_length_eq_one (n : ℕ) : n.primeFactorsList.length = 1 ↔ n.Prime
```
[](https://gitpod.io/from-referrer/)
|
t-data |
21/3 |
Mathlib/Data/Nat/Factors.lean |
1 |
5 |
['Ruben-VandeVelde', 'github-actions', 'qawbecrdtey'] |
nobody |
19-12667 19 days ago |
33-63494 1 month ago |
33-72095 33 days |
26483 |
metakunt author:metakunt |
feat (RingTheory/RootsOfUnity/PrimitiveRoots) : Add equiv_primitiveRoots_of_coprimePow |
Adds equivalence of r-th primitive roots by a coprime e. |
new-contributor
t-algebra
label:t-algebra$ |
79/0 |
Mathlib/RingTheory/RootsOfUnity/PrimitiveRoots.lean |
1 |
6 |
['Citronhat', 'github-actions', 'metakunt'] |
nobody |
19-9865 19 days ago |
22-26225 22 days ago |
22-26269 22 days |
26555 |
Komyyy author:Komyyy |
feat: lemmas about betweeness on a linear space |
This PR also adds aliases of the inverse direction of betweeness iff lemmas.
---
[](https://gitpod.io/from-referrer/)
|
t-euclidean-geometry |
86/0 |
Mathlib/Analysis/Convex/Between.lean |
1 |
1 |
['github-actions'] |
nobody |
19-6903 19 days ago |
19-34898 19 days ago |
19-38106 19 days |
26594 |
metakunt author:metakunt |
feat(Algebra/Polynomial/ZMod): Add Polynomial.equiv_of_nat_of_polynomial_zmod |
This adds an explicit bijection between the naturals and $$\mathbb{Z}/n\mathbb{Z}[X]$$ in a canonical way.
---
I feel that some API is missing to make the theorem shorter, I have no idea what lemmas to extract though.
Also I don't know when to use spaces and when not, so I did it best effort.
|
new-contributor
t-algebra
label:t-algebra$ |
465/0 |
Mathlib.lean,Mathlib/Algebra/Polynomial/ZMod.lean |
2 |
1 |
['github-actions'] |
nobody |
18-35904 18 days ago |
18-36934 18 days ago |
18-36981 18 days |
24917 |
adomani author:adomani |
feat: deprecated module automation |
This PR is a revised version of #24861. It splits the `#create_deprecated_modules` into two commands:
* `#create_deprecated_module path/to/file.lean` that guides you through generating a deprecated file;
* `#find_deleted_files n` that looks at the repository `n` commits ago and returns a `#create_deprecated_module` for each file that existed then and does not exist now.
This is integrated with `Try these:` suggestions and is intended as a first step in making this process completely automatic.
Each regenerated file consists of just the imports of the last file that existed, before deletion, followed by `deprecated_import (since := "YYYY-MM-DD")`.
In particular, this also applies to *renames*, where it might be more natural to suggest the renamed file, rather than its imports. However, this is part of the deprecation logic that I consider best left to a possible future PR, since distinguishing renames from removals is a separate matter that even git does not handle completely satisfactorily.
---
[](https://gitpod.io/from-referrer/)
|
t-meta |
381/0 |
scripts/README.md,scripts/create_deprecated_modules.lean |
2 |
47 |
['YaelDillies', 'adomani', 'github-actions', 'grunweg', 'leanprover-community-bot-assistant'] |
grunweg assignee:grunweg |
18-34973 18 days ago |
18-34994 18 days ago |
39-61634 39 days |
25841 |
mitchell-horner author:mitchell-horner |
feat(Combinatorics/SimpleGraph): prove the Kővári–Sós–Turán theorem |
Prove the Kővári–Sós–Turán theorem for simple graphs: the `(completeBipartiteGraph α β).Free` simple graphs for `card α ≤ card β` on the vertex type `V` have at most `(card β-1)^(1/(card α))*(card V)^(2-1/(card α))/2 + (card V)*(card α-1)/2` edges.
---
- [x] depends on: #19865
- [x] depends on: #20738
I'd like to make `aux` not private in the `KovariSosTuran` namespace to enable reuse of the double-counting here, but I don't know what to call it.
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #20240.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/20240* |
t-combinatorics |
289/0 |
Mathlib.lean,Mathlib/Combinatorics/SimpleGraph/Bipartite.lean,Mathlib/Combinatorics/SimpleGraph/Extremal/KovariSosTuran.lean |
3 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
awainverse assignee:awainverse |
18-30303 18 days ago |
36-52844 1 month ago |
36-52889 36 days |
25843 |
mitchell-horner author:mitchell-horner |
feat(Combinatorics/SimpleGraph): define `between` subgraphs |
The simple graph `G.between s t` is the subgraph of `G` containing edges that connect a vertex in the set `s` to a vertex in the set `t`.
---
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #24948.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/24948* |
t-combinatorics |
95/0 |
Mathlib/Combinatorics/SimpleGraph/Bipartite.lean |
1 |
1 |
['github-actions'] |
nobody |
18-30272 18 days ago |
36-52446 1 month ago |
36-52430 36 days |
25758 |
YaelDillies author:YaelDillies |
chore: shortcut instance `CompleteLattice α → PartialOrder α` |
This avoids using the path `CompleteLattice α → CompletePartialOrder α → PartialOrder α` that goes through `Order.CompletePartialOrder` and makes it appear used to our automation, such as `shake` or `#min_imports`.
This is a followup to #25358.
---
[](https://gitpod.io/from-referrer/)
|
t-order |
7/0 |
Mathlib/Order/CompleteLattice/Defs.lean |
1 |
6 |
['Ruben-VandeVelde', 'eric-wieser', 'github-actions', 'leanprover-bot'] |
nobody |
18-17410 18 days ago |
18-19435 18 days ago |
37-70020 37 days |
25715 |
kbuzzard author:kbuzzard |
feat: more RestrictedProduct API |
A constructor, more algebra boilerplate (e.g. `SMul ℕ` on a restricted product of `AddMonoid`s, restricted product of `CommMonoid`s is a `CommMonoid`, restricted product of `R`-modules wrt `R`-submodules is an `R`-module, variant of `map` when the index set doesn't change.
From the FLT project.
---
[](https://gitpod.io/from-referrer/)
|
FLT
t-topology
|
91/36 |
Mathlib/Topology/Algebra/RestrictedProduct/Basic.lean |
1 |
13 |
['ADedecker', 'github-actions', 'kbuzzard', 'matthewjasper'] |
nobody |
18-14663 18 days ago |
38-17521 1 month ago |
38-21321 38 days |
25989 |
Multramate author:Multramate |
feat(NumberTheory/EllipticDivisibilitySequence): add elliptic nets |
This PR continues the work from #25030.
Original PR: https://github.com/leanprover-community/mathlib4/pull/25030 |
t-number-theory |
259/37 |
Mathlib/NumberTheory/EllipticDivisibilitySequence.lean |
1 |
3 |
['MichaelStollBayreuth', 'Multramate', 'github-actions'] |
nobody |
17-34833 17 days ago |
33-21463 1 month ago |
33-21509 33 days |
26638 |
metakunt author:metakunt |
chore: Add grind to cast_zero |
Add grind to cast_zero |
t-data
new-contributor
|
1/1 |
Mathlib/Data/Nat/Cast/Defs.lean |
1 |
1 |
['github-actions'] |
nobody |
17-32282 17 days ago |
17-32282 17 days ago |
17-33885 17 days |
26563 |
winstonyin author:winstonyin |
chore: rename `IsIntegralCurve` to `IsMIntegralCurve` |
I rename all the existing `IsIntegralCurve` series of definitions and lemmas for manifolds to `IsMIntegralCurve` in preparation for reusing `IsIntegralCurve` for the vector space version.
- [ ] depends on: #26533
---
[](https://gitpod.io/from-referrer/)
|
t-differential-geometry |
320/165 |
Mathlib/Geometry/Manifold/IntegralCurve/Basic.lean,Mathlib/Geometry/Manifold/IntegralCurve/ExistUnique.lean,Mathlib/Geometry/Manifold/IntegralCurve/Transform.lean,Mathlib/Geometry/Manifold/IntegralCurve/UniformTime.lean,docs/overview.yaml |
5 |
8 |
['github-actions', 'grunweg', 'mathlib4-dependent-issues-bot', 'winstonyin'] |
grunweg assignee:grunweg |
17-19308 17 days ago |
17-19487 17 days ago |
17-58909 17 days |
23986 |
ShouxinZhang author:ShouxinZhang |
feat(FieldTheory/RatFunc): add RatFunc.toFractionRingAlgEquiv |
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-algebra
label:t-algebra$ |
13/0 |
Mathlib/FieldTheory/RatFunc/Basic.lean |
1 |
32 |
['ShouxinZhang', 'eric-wieser', 'github-actions', 'joneugster', 'kckennylau', 'plp127'] |
nobody |
17-12990 17 days ago |
19-25846 19 days ago |
98-2384 98 days |
26370 |
b-mehta author:b-mehta |
chore(Archive): golf and generalise ascending-descending sequences |
This proof was 5 years old, not in a good generality, and overly long. We fix the latter two points.
---
[](https://gitpod.io/from-referrer/)
|
t-data |
96/120 |
Archive/Wiedijk100Theorems/AscendingDescendingSequences.lean |
1 |
12 |
['b-mehta', 'github-actions', 'grunweg'] |
nobody |
17-6508 17 days ago |
23-64453 23 days ago |
25-32991 25 days |
26148 |
Hagb author:Hagb |
feat(RingTheory/Ideal/Span): some lemmas about zero and span |
`simp` would be able to solve them.
Notice that `span_singleton_zero : span {(0 : R)} = ⊥` itself can be solved by `simp` without this commit, which uses `span_singleton_eq_bot : span ({x} : Set α) = ⊥ ↔ x = 0`, while `simp` cannot solve goals like `f (Ideal.span {(0 : R)}) = f ⊥`, which would be solvable by `simp` with `span_singleton_zero` marked with `@[simp]`.
Without adding also `Ideal.dvd_bot`, these lemmas on `Span.lean` would make the following failed, since `simp` would rewrite `{0}` with `⊥` and result in a goal `v.asIdeal ∣ ⊥` that it can't solve.
https://github.com/leanprover-community/mathlib4/blob/3f2556372f27171259a381d4d57db71440700cd8/Mathlib/RingTheory/DedekindDomain/AdicValuation.lean#L123
---
This PR continues the work from #24448.
Original PR: #24448.
CC: @tb65536
[](https://gitpod.io/from-referrer/)
|
migrated-from-branch
t-algebra
label:t-algebra$ |
11/0 |
Mathlib/RingTheory/Ideal/Operations.lean,Mathlib/RingTheory/Ideal/Span.lean |
2 |
1 |
['github-actions'] |
nobody |
16-76524 16 days ago |
16-76524 16 days ago |
30-62042 30 days |
26645 |
erdOne author:erdOne |
feat(RingTheory/PowerSeries): Construction of `Q` such that `P(Q(X)) = X` |
Co-authored-by: Junnosuke Koizumi
Co-authored-by: Hyeon, Seung-Hyeon
Co-authored-by: Yuichiro Taguchi
This contribution was created as part of the ZMC conference 2025 "Anabelian Geometry and its Computer Formalization".
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
133/0 |
Mathlib/RingTheory/PowerSeries/Substitution.lean |
1 |
9 |
['chrisflav', 'erdOne', 'github-actions', 'kckennylau'] |
nobody |
16-65765 16 days ago |
17-15365 17 days ago |
17-15411 17 days |
26378 |
EtienneC30 author:EtienneC30 |
feat: inner product against funBasis |
Also remove the `simp` attribute off [PiLp.inner_apply](https://leanprover-community.github.io/mathlib4_docs/Mathlib/Analysis/InnerProductSpace/PiL2.html#PiLp.inner_apply).
---
[](https://gitpod.io/from-referrer/)
|
t-analysis |
17/7 |
Mathlib/Analysis/InnerProductSpace/PiL2.lean,Mathlib/Analysis/RCLike/Inner.lean |
2 |
4 |
['EtienneC30', 'eric-wieser', 'github-actions'] |
nobody |
16-59050 16 days ago |
18-61752 18 days ago |
25-23287 25 days |
22039 |
YaelDillies author:YaelDillies |
feat: simproc for computing `Finset.Ixx` of natural numbers |
---
- [x] depends on: #22290
- [x] depends on: #22559
[](https://gitpod.io/from-referrer/)
|
large-import
t-meta
|
315/0 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Simproc/FinsetInterval.lean,Mathlib/Util/Qq.lean |
4 |
59 |
['FLDutchmann', 'Paul-Lez', 'YaelDillies', 'eric-wieser', 'github-actions', 'grunweg', 'kim-em', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'urkud'] |
eric-wieser assignee:eric-wieser |
16-51416 16 days ago |
94-64799 3 months ago |
150-25518 150 days |
26313 |
kckennylau author:kckennylau |
feat: 4 lemmas about Finsupp.mapDomain.linearEquiv |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
9/0 |
Mathlib/LinearAlgebra/Finsupp/Defs.lean |
1 |
5 |
['eric-wieser', 'github-actions', 'kckennylau'] |
nobody |
16-41620 16 days ago |
26-43141 26 days ago |
26-43192 26 days |
26192 |
kckennylau author:kckennylau |
feat(LinearAlgebra): symmetric tensor power |
---
Zulip: [#mathlib4 > Proposal: Symmetric Tensor Power](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Proposal.3A.20Symmetric.20Tensor.20Power/with/524795235)
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
129/0 |
Mathlib.lean,Mathlib/LinearAlgebra/TensorPower/Symmetric.lean |
2 |
6 |
['AntoineChambert-Loir', 'erdOne', 'eric-wieser', 'github-actions', 'kckennylau'] |
nobody |
16-40709 16 days ago |
30-15374 1 month ago |
30-15418 30 days |
26694 |
BoltonBailey author:BoltonBailey |
feat: add lemmas for modular exponentiation with the totient function |
This PR adds lemmas around reducing the exponent of a modular exponentiation.
These lemmas were found while doing work for [Project Numina](https://projectnumina.ai/).
---
[](https://gitpod.io/from-referrer/)
|
t-data |
51/0 |
Mathlib.lean,Mathlib/Data/Nat/PowModTotient.lean |
2 |
1 |
['github-actions'] |
nobody |
16-31446 16 days ago |
16-36233 16 days ago |
16-36278 16 days |
25692 |
Whysoserioushah author:Whysoserioushah |
feat(RingTheory/MatrixAlgebra): add a more general version of `matrixEquivTensor` |
This adds `tensorMatrixLinearEquiv : A ⊗[R] Matrix n n B ≃ₐ[S] Matrix n n (A ⊗[R] B)`
which is a more general version of `matrixEquivTensor : Matrix n n A ≃ₐ[R] (A ⊗[R] Matrix n n R)`.
The latter is then implemented as a trivial consequence of the former.
Many internal implementation details are deleted without deprecation, although strictly these were not `private.
Co-authored-by: @erdOne
Co-authored-by: Eric Wieser
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
122/100 |
Mathlib/Data/Matrix/Basis.lean,Mathlib/RingTheory/MatrixAlgebra.lean |
2 |
13 |
['Whysoserioushah', 'eric-wieser', 'github-actions'] |
nobody |
16-26253 16 days ago |
22-10741 22 days ago |
38-66544 38 days |
26670 |
yu-yama author:yu-yama |
feat(GroupExtension/Abelian): define `conjClassesEquivH1` |
This PR continues the work from #21837.
Original PR: https://github.com/leanprover-community/mathlib4/pull/21837 |
t-algebra label:t-algebra$ |
162/5 |
Mathlib.lean,Mathlib/GroupTheory/GroupExtension/Abelian.lean,Mathlib/GroupTheory/GroupExtension/Basic.lean,Mathlib/GroupTheory/GroupExtension/Defs.lean,docs/references.bib |
5 |
2 |
['erdOne', 'github-actions', 'yu-yama'] |
nobody |
16-17514 16 days ago |
16-46019 16 days ago |
16-46071 16 days |
26710 |
metakunt author:metakunt |
feat (Data/Nat/Digits/Lemmas): Add digits_getD |
Adds digits_getD, an explicit computation of the i-th digits of n in base b representation. |
t-data
new-contributor
|
64/0 |
Mathlib/Data/Nat/Digits/Lemmas.lean |
1 |
1 |
['github-actions'] |
nobody |
16-14937 16 days ago |
16-15068 16 days ago |
16-15120 16 days |
24064 |
kim-em author:kim-em |
chore: replace `norm_num` with `simp` where applicable |
Consider replacing a tactic with a (ahem) simpler alternative.
Fairly neutral performance implications, just depends on whether we would like to encourage people to use `simp` where applicable. |
|
336/336 |
Archive/Examples/MersennePrimes.lean,Archive/Imo/Imo1959Q2.lean,Archive/Imo/Imo1960Q1.lean,Archive/Imo/Imo1962Q1.lean,Archive/Imo/Imo1962Q4.lean,Archive/Imo/Imo1981Q3.lean,Archive/Imo/Imo1982Q1.lean,Archive/Imo/Imo2001Q2.lean,Archive/Imo/Imo2005Q4.lean,Archive/Imo/Imo2006Q3.lean,Archive/Imo/Imo2008Q4.lean,Archive/Imo/Imo2024Q1.lean,Archive/Imo/Imo2024Q5.lean,Archive/Imo/Imo2024Q6.lean,Archive/Wiedijk100Theorems/AbelRuffini.lean,Archive/Wiedijk100Theorems/CubingACube.lean,Archive/Wiedijk100Theorems/SumOfPrimeReciprocalsDiverges.lean,Counterexamples/Cyclotomic105.lean,Counterexamples/Phillips.lean,Mathlib/Algebra/Field/NegOnePow.lean,Mathlib/Algebra/Homology/HomotopyCategory/MappingCone.lean,Mathlib/Algebra/Order/CauSeq/BigOperators.lean,Mathlib/Algebra/Polynomial/FieldDivision.lean,Mathlib/Algebra/Polynomial/Roots.lean,Mathlib/Algebra/Polynomial/SpecificDegree.lean,Mathlib/Algebra/Ring/BooleanRing.lean,Mathlib/Algebra/Star/CHSH.lean,Mathlib/AlgebraicGeometry/EllipticCurve/IsomOfJ.lean,Mathlib/AlgebraicTopology/DoldKan/Faces.lean,Mathlib/Analysis/Analytic/Inverse.lean,Mathlib/Analysis/Asymptotics/AsymptoticEquivalent.lean,Mathlib/Analysis/BoxIntegral/UnitPartition.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Basic.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Order.lean,Mathlib/Analysis/CStarAlgebra/Module/Defs.lean,Mathlib/Analysis/Calculus/FDeriv/Measurable.lean,Mathlib/Analysis/Calculus/FDeriv/Norm.lean,Mathlib/Analysis/Calculus/FDeriv/Symmetric.lean,Mathlib/Analysis/Complex/AbelLimit.lean,Mathlib/Analysis/Convex/Between.lean,Mathlib/Analysis/Convex/Function.lean,Mathlib/Analysis/Convolution.lean,Mathlib/Analysis/Fourier/AddCircle.lean,Mathlib/Analysis/Fourier/AddCircleMulti.lean,Mathlib/Analysis/Fourier/Inversion.lean,Mathlib/Analysis/Fourier/RiemannLebesgueLemma.lean,Mathlib/Analysis/InnerProductSpace/NormPow.lean,Mathlib/Analysis/InnerProductSpace/Projection.lean,Mathlib/Analysis/InnerProductSpace/l2Space.lean,Mathlib/Analysis/MeanInequalities.lean,Mathlib/Analysis/MellinInversion.lean,Mathlib/Analysis/Normed/Affine/Simplex.lean,Mathlib/Analysis/Normed/Algebra/TrivSqZeroExt.lean,Mathlib/Analysis/Normed/Group/ControlledClosure.lean,Mathlib/Analysis/Normed/Lp/lpSpace.lean,Mathlib/Analysis/Normed/Operator/Banach.lean,Mathlib/Analysis/Normed/Ring/Units.lean,Mathlib/Analysis/NormedSpace/HahnBanach/Separation.lean,Mathlib/Analysis/NormedSpace/MStructure.lean,Mathlib/Analysis/NormedSpace/RieszLemma.lean,Mathlib/Analysis/Oscillation.lean,Mathlib/Analysis/SpecialFunctions/BinaryEntropy.lean,Mathlib/Analysis/SpecialFunctions/Complex/Log.lean,Mathlib/Analysis/SpecialFunctions/ContinuousFunctionalCalculus/Rpow/Basic.lean,Mathlib/Analysis/SpecialFunctions/ContinuousFunctionalCalculus/Rpow/Isometric.lean,Mathlib/Analysis/SpecialFunctions/ExpDeriv.lean,Mathlib/Analysis/SpecialFunctions/Gamma/Beta.lean,Mathlib/Analysis/SpecialFunctions/Gamma/BohrMollerup.lean,Mathlib/Analysis/SpecialFunctions/Gamma/Deligne.lean,Mathlib/Analysis/SpecialFunctions/Gaussian/GaussianIntegral.lean,Mathlib/Analysis/SpecialFunctions/Integrals/Basic.lean,Mathlib/Analysis/SpecialFunctions/Log/Monotone.lean,Mathlib/Analysis/SpecialFunctions/Pow/Real.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Angle.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Basic.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Complex.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Inverse.lean,Mathlib/Combinatorics/Additive/AP/Three/Behrend.lean,Mathlib/Combinatorics/Additive/SmallTripling.lean,Mathlib/Combinatorics/Extremal/RuzsaSzemeredi.lean,Mathlib/Combinatorics/SimpleGraph/Density.lean,Mathlib/Combinatorics/SimpleGraph/Regularity/Bound.lean,Mathlib/Combinatorics/SimpleGraph/Regularity/Chunk.lean,Mathlib/Combinatorics/SimpleGraph/Regularity/Increment.lean,Mathlib/Combinatorics/SimpleGraph/Regularity/Lemma.lean,Mathlib/Combinatorics/SimpleGraph/Triangle/Basic.lean,Mathlib/Combinatorics/SimpleGraph/Triangle/Counting.lean,Mathlib/Computability/Ackermann.lean,Mathlib/Computability/DFA.lean,Mathlib/Data/Complex/Basic.lean,Mathlib/Data/Complex/Trigonometric.lean,Mathlib/Data/Nat/Bits.lean,Mathlib/Data/Nat/Choose/Central.lean,Mathlib/Data/Nat/Choose/Sum.lean,Mathlib/Data/Nat/Digits/Defs.lean,Mathlib/Data/Nat/Prime/Defs.lean,Mathlib/Data/Real/GoldenRatio.lean,Mathlib/Data/Real/Pi/Bounds.lean,Mathlib/Data/Real/Pi/Irrational.lean,Mathlib/Data/Real/Sign.lean |
170 |
9 |
['github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'leanprover-community-mathlib4-bot'] |
nobody |
16-8692 16 days ago |
16-8710 16 days ago |
27-74342 27 days |
25812 |
vlad902 author:vlad902 |
feat(data): List.Chain' helper lemmas |
Add two helpers lemmas to go from a List.Chain' hypothesis to a concrete
predicate about two consecutive elements, one in the positive and one in
the negative. |
t-data |
29/0 |
Mathlib/Data/List/Chain.lean |
1 |
4 |
['BoltonBailey', 'github-actions', 'vlad902'] |
nobody |
15-82205 15 days ago |
16-70499 16 days ago |
29-73087 29 days |
26267 |
vasnesterov author:vasnesterov |
feat(Analysis/Calculus): Taylor series converges to function on whole ball |
* Prove `FormalMultilinearSeries.AnalyticOnNhd`: the sum of series is analytic on its ball of convergence.
* Prove `AnalyticOn.hasFPowerSeriesOnBall`: a variant of `AnalyticAt.hasFPowerSeriesAt` which gives convergence to the function on the ball of convergence.
---
- [x] depends on: #23745
- [x] depends on: #23747
- [x] depends on: #23748
- [x] depends on: #26247
This PR continues the work from #23749.
Original PR: https://github.com/leanprover-community/mathlib4/pull/23749 |
large-import
t-analysis
|
47/0 |
Mathlib/Analysis/Analytic/ChangeOrigin.lean,Mathlib/Analysis/Calculus/IteratedDeriv/Lemmas.lean |
2 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'vasnesterov'] |
nobody |
15-80750 15 days ago |
16-3846 16 days ago |
16-10160 16 days |
26597 |
sahanwijetunga author:sahanwijetunga |
Update Orthogonal.lean |
fixed documentation for orthogonal (regarding order of inputs to bilinear form)
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-algebra
documentation
label:t-algebra$ |
3/3 |
Mathlib/LinearAlgebra/BilinearForm/Orthogonal.lean |
1 |
2 |
['github-actions', 'mbkybky'] |
nobody |
15-77491 15 days ago |
15-77498 15 days ago |
18-29965 18 days |
26037 |
joelriou author:joelriou |
feat(Order): bicartesian squares in lattices |
This PR introduces the notion of bicartesian square in lattices (and a more general "multicoequalizer" version in complete lattices). In the case of the lattice `Set X`, this will give respectively bicartesian squares (both pushout and pullback) and multicoequalizer diagrams in the category of sets.
---
- [x] depends on: #22203
- [x] depends on: #26028
- [x] depends on: #20988
This PR continues the work from #21032.
Original PR: https://github.com/leanprover-community/mathlib4/pull/21032 |
t-order
t-category-theory
|
116/0 |
Mathlib.lean,Mathlib/Order/CompleteLattice/MulticoequalizerDiagram.lean |
2 |
3 |
['github-actions', 'joelriou', 'mathlib4-dependent-issues-bot'] |
nobody |
15-72512 15 days ago |
15-72512 15 days ago |
16-907 16 days |
25179 |
YaelDillies author:YaelDillies |
feat: `#print sorries`, a command to find usage of `sorry` |
`#print sorries` returns all sorries in the current file. `#print sorries id1 ... idn` returns all sorries in declarations `id1`, ..., `idn`.
Such a command is a recurrent need of the community, see eg [here](https://leanprover.zulipchat.com/#narrow/channel/217875-Is-there-code-for-X.3F/topic/Hunting.20down.20axioms/with/495448595) most recently.
From Toric
Co-authored-by: Henrik Böving
Co-authored-by: Kyle Miller
---
An alternative implementation was provided in [#Is there code for X? > ✔ Finding usages of `sorry` in external code @ 💬](https://leanprover.zulipchat.com/#narrow/channel/217875-Is-there-code-for-X.3F/topic/.E2.9C.94.20Finding.20usages.20of.20.60sorry.60.20in.20external.20code/near/430509619) by @kmill. I prefer the current one because it only prints something for uses of `sorry` and not the other three standard axioms.
[](https://gitpod.io/from-referrer/)
|
toric
t-meta
|
103/0 |
Mathlib.lean,Mathlib/Util/PrintSorries.lean |
2 |
11 |
['YaelDillies', 'eric-wieser', 'github-actions', 'kmill'] |
nobody |
15-68497 15 days ago |
55-71244 1 month ago |
55-71295 55 days |
26000 |
Hagb author:Hagb |
feat(RingTheory/MvPolynomial/MonomialOrder): some lemmas about degree |
Co-authored-by: Hao Shen @tsuki8 <3118181069@qq.com>
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
24/0 |
Mathlib/RingTheory/MvPolynomial/MonomialOrder.lean |
1 |
6 |
['Hagb', 'Ruben-VandeVelde', 'github-actions'] |
nobody |
15-51097 15 days ago |
15-51644 15 days ago |
29-57824 29 days |
24794 |
chrisflav author:chrisflav |
feat(RingTheory/Presentation): core of a presentation |
If `P` is a presentation of `S` as an `R`-algebra and `R₀` a subring of `R` containing the coefficients of the relations of `P`, then there exists an `R₀`-algebra `S₀` such that `S` is isomorphic to the base change of `S₀` to `R`.
This is a tool to remove Noetherian hypothesis in certain situations.
---
- [x] depends on: #24788
- [x] depends on: #24786
- [x] depends on: #24785
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
252/2 |
Mathlib.lean,Mathlib/Algebra/Algebra/Subalgebra/Basic.lean,Mathlib/Algebra/Algebra/Subalgebra/Tower.lean,Mathlib/Algebra/Algebra/Tower.lean,Mathlib/RingTheory/AlgebraicIndependent/Transcendental.lean,Mathlib/RingTheory/Extension/Presentation/Core.lean,Mathlib/RingTheory/FiniteType.lean,Mathlib/RingTheory/TensorProduct/MvPolynomial.lean |
8 |
10 |
['erdOne', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
15-46393 15 days ago |
40-71550 1 month ago |
40-72488 40 days |
26759 |
MichaelStollBayreuth author:MichaelStollBayreuth |
chore(Algebra/Polynomial/IsMonicOfDegree): do not import compute_degree tactic |
To prepare for an extension of the `monicity` tactic to also work for `IsMonicOfDegree`, avoid importing this and related tactics in the file that defines `IsMonicOfDegree`.
This means that some proof that used `compute_degree` or `compute_degree!` need to be spelled out in terms of the API for `Polynomial.natDegree`.
Zulip: [#mathlib4 > Gelfand-Mazur theorem @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Gelfand-Mazur.20theorem/near/526268507)
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
15/8 |
Mathlib/Algebra/Polynomial/Degree/IsMonicOfDegree.lean |
1 |
1 |
['github-actions'] |
nobody |
15-39771 15 days ago |
15-39771 15 days ago |
15-39754 15 days |
26766 |
MichaelStollBayreuth author:MichaelStollBayreuth |
feat(Topology/MetricSpace/Bounded): add some results |
We add two pairs of results:
```lean
lemma isBounded_of_abs_le (C : α) : Bornology.IsBounded {x : α | |x| ≤ C} := ...
lemma isBounded_of_abs_lt (C : α) : Bornology.IsBounded {x : α | |x| < C} := ...
```
(under suitable assumptions on `α`) and a version of the *Extreme Value Theorem* that I found convenient:
```lean
theorem exists_forall_le_of_isBounded {f : β → α} (hf : Continuous f) (x₀ : β)
(h : Bornology.IsBounded {x : β | f x ≤ f x₀}) :
∃ x, ∀ y, f x ≤ f y := ...
theorem exists_forall_ge_of_isBounded {f : β → α} (hf : Continuous f) (x₀ : β)
(h : Bornology.IsBounded {x : β | f x₀ ≤ f x}) :
∃ x, ∀ y, f y ≤ f x := ...
```
(under suitable assumptions on `α` and `β`).
For an application, see [GelfandMazur.lean](https://github.com/MichaelStollBayreuth/Heights/blob/master/Heights/GelfandMazur.lean) in [Heights](https://github.com/MichaelStollBayreuth/Heights/tree/master).
---
[](https://gitpod.io/from-referrer/)
|
t-topology |
56/0 |
Mathlib/Topology/MetricSpace/Bounded.lean |
1 |
1 |
['github-actions'] |
nobody |
15-31744 15 days ago |
15-31744 15 days ago |
15-31727 15 days |
25889 |
plp127 author:plp127 |
fix(Tactic/Widget/Conv): fix various issues |
Fixes various issues with the `conv?` widget. Closes #25162.
([Zulip thread](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/bug.20in.20.60conv.3F.60))
Specifically, fixes issues with `conv?` where
- when converting a `SubExpr.Pos` to conv directions, it always uses the goal expression as reference, even when working on a hypothesis, this often leads to bad results and makes it unusable on hypotheses
- it refuses to go all the way in to a function (for example in `Nat.succ 0`, you can't access `Nat.succ`)
- it refuses to enter binders where the name of the bound variable contains the character `0` (try it on `∀ (x0 : Nat), x0 = x0`)
- it panics if it can't find a binder name instead of just coming up with one itself, this also means usually you can't enter either side of a non-dependent arrow since those usually don't have binder names (try it on `False → False`)
- you can't enter the type of a binder, you end up going into the body instead (try it on `fun (x : False) => (x.elim : False → Nat) x.elim`)
- you can't partially enter a function, you end up going to the top argument after instead (for example, in the expression `id (id id) 0`, when you click on `id (id id)`, you end up going to `id id`)
---
[](https://gitpod.io/from-referrer/)
|
t-meta |
110/83 |
Mathlib/Tactic/Widget/Conv.lean |
1 |
4 |
['bryangingechen', 'github-actions', 'plp127'] |
nobody |
15-1533 15 days ago |
35-5317 1 month ago |
35-5362 35 days |
19872 |
YaelDillies author:YaelDillies |
chore(GroupTheory/Index): rename `relindex` to `relIndex` |
---
- [x] depends on: #24044
[](https://gitpod.io/from-referrer/)
|
FLT
t-algebra
label:t-algebra$ |
257/194 |
Mathlib/FieldTheory/Relrank.lean,Mathlib/GroupTheory/Commensurable.lean,Mathlib/GroupTheory/CosetCover.lean,Mathlib/GroupTheory/GroupAction/Blocks.lean,Mathlib/GroupTheory/Index.lean,Mathlib/GroupTheory/IndexNormal.lean,Mathlib/GroupTheory/PGroup.lean,Mathlib/GroupTheory/Schreier.lean,Mathlib/GroupTheory/SchurZassenhaus.lean,Mathlib/GroupTheory/Sylow.lean,Mathlib/GroupTheory/Transfer.lean,Mathlib/LinearAlgebra/FreeModule/Finite/CardQuotient.lean,Mathlib/NumberTheory/ModularForms/CongruenceSubgroups.lean,Mathlib/NumberTheory/NumberField/Discriminant/Different.lean,Mathlib/NumberTheory/NumberField/Units/Regulator.lean,Mathlib/RingTheory/Ideal/Quotient/Index.lean |
16 |
24 |
['Ruben-VandeVelde', 'TwoFX', 'YaelDillies', 'alreadydone', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'loefflerd', 'madvorak', 'mathlib4-dependent-issues-bot', 'tb65536'] |
nobody |
14-76986 14 days ago |
14-79568 14 days ago |
169-30498 169 days |
25732 |
robin-carlier author:robin-carlier |
feat(CategoryTheory/Monoidal/Limits): miscellany about preservation of (co)limits by tensor products |
Register some instances regarding preservations of (co)limits for the tensor product of a monoidal category. More precisely, we register the fact that if the category is braided and `tensorLeft c` preserves colimits (this can be inferred e.g via `MonoidalClosed C`), then so does `tensorRight c` for every `c`.
We also rephrase preservation of (co)limits for `curriedTensor C` in terms of preservations of (co)limits for `tensorRight c`.
The PR introduces also introduces a directory `CategoryTheory.Monoidal.Limits` and moves the existing file `CategoryTheory.Monoidal.Limits.lean` to `CategoryTheory.Monoidal.Limits.Basic`.
---
The instances registered here are tailored so that for a braided monoidal closed category, `PreservesColimit₂` instances from #24685 can be inferred with the results of #24686 for the external product of diagrams defined in #24703
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #24711.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/24711* |
file-removed
t-category-theory
|
72/2 |
Mathlib.lean,Mathlib/CategoryTheory/Monoidal/Internal/Limits.lean,Mathlib/CategoryTheory/Monoidal/Limits/Basic.lean,Mathlib/CategoryTheory/Monoidal/Limits/Preserves.lean |
4 |
2 |
['github-actions', 'leanprover-community-bot-assistant'] |
nobody |
14-76814 14 days ago |
14-76832 14 days ago |
37-66017 37 days |
22655 |
YaelDillies author:YaelDillies |
refactor: make use of `FunLike` for `Submonoid.LocalizationMap` |
From Toric
---
[](https://gitpod.io/from-referrer/)
|
toric
t-algebra
label:t-algebra$ |
161/146 |
Mathlib/GroupTheory/MonoidLocalization/Away.lean,Mathlib/GroupTheory/MonoidLocalization/Basic.lean,Mathlib/GroupTheory/MonoidLocalization/DivPairs.lean,Mathlib/GroupTheory/MonoidLocalization/MonoidWithZero.lean,Mathlib/RingTheory/Localization/Defs.lean,Mathlib/RingTheory/Valuation/ExtendToLocalization.lean |
6 |
4 |
['github-actions', 'leanprover-community-bot-assistant'] |
ericrbg assignee:ericrbg |
14-76349 14 days ago |
14-76371 14 days ago |
131-66990 131 days |
26110 |
YaelDillies author:YaelDillies |
feat: sharp monoids |
Define sharp monoids, which are the monoids whose only unit is `1`. This concept is useful in log geometry and in particular shows up in the theory of affine monoids.
This concept already existed in the guise of `Subsingleton Mˣ`, but giving it a name makes it easier to refer to and uncovers some missing instances.
From Toric
---
[](https://gitpod.io/from-referrer/)
|
toric
t-algebra
label:t-algebra$ |
51/30 |
Mathlib/Algebra/BigOperators/Associated.lean,Mathlib/Algebra/BigOperators/Group/Finset/Basic.lean,Mathlib/Algebra/GCDMonoid/Basic.lean,Mathlib/Algebra/Group/Irreducible/Defs.lean,Mathlib/Algebra/Group/Pi/Units.lean,Mathlib/Algebra/Group/Prod.lean,Mathlib/Algebra/Group/Submonoid/Units.lean,Mathlib/Algebra/Group/Units/Basic.lean,Mathlib/Algebra/Group/Units/Defs.lean,Mathlib/Algebra/GroupWithZero/Associated.lean,Mathlib/Algebra/GroupWithZero/Divisibility.lean,Mathlib/Data/List/Prime.lean,Mathlib/Data/ZMod/Basic.lean,Mathlib/NumberTheory/DirichletCharacter/Basic.lean,Mathlib/RingTheory/ChainOfDivisors.lean,Mathlib/RingTheory/IntegralDomain.lean,Mathlib/RingTheory/UniqueFactorizationDomain/NormalizedFactors.lean,Mathlib/RingTheory/Valuation/Integers.lean |
18 |
2 |
['b-mehta', 'github-actions', 'leanprover-community-bot-assistant'] |
nobody |
14-75784 14 days ago |
14-81064 14 days ago |
31-40714 31 days |
26021 |
vasnesterov author:vasnesterov |
feat(Data/Real): representation of reals from `[0, 1]` in positional system |
* Introduce `ofDigits {b : ℕ} (digits : ℕ → Fin b) : ℝ`, representing a real number of the form `0.d₀d₁d₂...` (where `dᵢ = digits i`) as an infinite sum.
* Prove that this sum converges to a number in the interval `[0, 1]`.
* Prove `ofDigits_close_of_common_prefix`: if the first `n` digits of two numbers are equal, then their difference is bounded by `b⁻ⁿ`.
* Introduce `Real.digits`, which converts a real number into its sequence of digits.
* Prove that `ofDigits (toDigits x b) = x`.
[Zulip thread](https://leanprover.zulipchat.com/#narrow/stream/217875-Is-there-code-for-X.3F/topic/Base.20n.20expansion.20of.20real.20numbers.3F/near/502937293)
---
- [x] depends on: #26004
[](https://gitpod.io/from-referrer/)
|
t-data |
238/0 |
Mathlib.lean,Mathlib/Data/Real/OfDigits.lean,scripts/noshake.json |
3 |
11 |
['alreadydone', 'eric-wieser', 'github-actions', 'mathlib4-dependent-issues-bot', 'vasnesterov', 'wwylele'] |
nobody |
14-73854 14 days ago |
18-2222 18 days ago |
18-2780 18 days |
26142 |
YaelDillies author:YaelDillies |
chore(GeomSum): split into ring vs field and non-ordered vs ordered parts |
The motivation here is that `Data.Nat.Multiplicity` needs the results about geometric sums of naturals, without wanting to know anything about fields.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
708/638 |
Archive/Imo/Imo1982Q3.lean,Archive/Imo/Imo2013Q5.lean,Archive/Wiedijk100Theorems/PerfectNumbers.lean,Counterexamples/ZeroDivisorsInAddMonoidAlgebras.lean,Mathlib.lean,Mathlib/Algebra/Field/GeomSum.lean,Mathlib/Algebra/GeomSum.lean,Mathlib/Algebra/Order/CauSeq/BigOperators.lean,Mathlib/Algebra/Order/Field/GeomSum.lean,Mathlib/Algebra/Order/Ring/GeomSum.lean,Mathlib/Algebra/Ring/GeomSum.lean,Mathlib/Analysis/Polynomial/CauchyBound.lean,Mathlib/Analysis/SpecificLimits/Basic.lean,Mathlib/Analysis/SpecificLimits/FloorPow.lean,Mathlib/Combinatorics/Colex.lean,Mathlib/Combinatorics/SetFamily/KruskalKatona.lean,Mathlib/Data/Nat/Multiplicity.lean,Mathlib/LinearAlgebra/Projectivization/Cardinality.lean,Mathlib/LinearAlgebra/Vandermonde.lean,Mathlib/NumberTheory/Basic.lean,Mathlib/NumberTheory/FactorisationProperties.lean,Mathlib/NumberTheory/MulChar/Basic.lean,Mathlib/NumberTheory/Multiplicity.lean,Mathlib/RingTheory/AdicCompletion/Basic.lean,Mathlib/RingTheory/Ideal/Quotient/Index.lean,Mathlib/RingTheory/Idempotents.lean,Mathlib/RingTheory/IntegralDomain.lean,Mathlib/RingTheory/Nilpotent/Basic.lean,Mathlib/RingTheory/Polynomial/Basic.lean,Mathlib/Tactic/NormNum/Irrational.lean |
30 |
2 |
['github-actions', 'leanprover-community-bot-assistant'] |
nobody |
14-73581 14 days ago |
14-80057 14 days ago |
30-57743 30 days |
26057 |
YaelDillies author:YaelDillies |
feat: `mon_tauto`, a simp set to prove tautologies about a monoid object |
This simp set proves all tautologies involving (commutative) monoid objects in a (braided) monoidal category.
The general algorithm it follows is to push the associators `α_` and commutators `β_` inwards until they cancel against the right sequence of multiplications.
This approach is justified by the fact that a tautology in the language of (commutative) monoid objects "remembers" how it was proved: Every use of a (commutative) monoid object axiom inserts a unitor, associator or commutator, and proving a tautology simply amounts to undoing those moves as prescribed by the presence of unitors, associators and commutators in its expression.
This simp set is opiniated about its normal form and therefore cannot be used concurrently to some of the simp lemmas in the standard simp set.
As an example, we prove `tensorμ M M M M ≫ (μ ⊗ₘ μ) ≫ μ = (μ ⊗ₘ μ) ≫ μ`, the categorical equivalent of `mul_mul_mul_comm`.
From Toric
Co-authored-by: Andrew Yang
---
- [x] depends on: #26102
[](https://gitpod.io/from-referrer/)
|
toric
t-category-theory
|
151/1 |
Mathlib/CategoryTheory/Monoidal/Mon_.lean,Mathlib/Tactic/Attr/Register.lean,MathlibTest/CategoryTheory/Monoidal/MonTauto.lean,scripts/noshake.json |
4 |
11 |
['YaelDillies', 'erdOne', 'github-actions', 'mathlib4-dependent-issues-bot', 'robin-carlier'] |
nobody |
14-73573 14 days ago |
31-30548 1 month ago |
32-7003 32 days |
25779 |
robin-carlier author:robin-carlier |
feat(CategoryTheory/Bicategory/NaturalTransformations): strong and lax natural transformations of lax functors |
Given two lax functors `F G` between bicategories, we define lax natural transformations as families of 1-morphisms `∀ a : B, F.obj a ⟶ G.obj a` equipped with a naturality 2-cell `∀ {a b : B} (f : a ⟶ b), app a ≫ G.map f ⟶ F.map f ≫ app b` that are required to satisfy conditions such as naturality, and compatibility with the `mapId` and `mapComp` fields of the source and target functors.
This notion dualizes the existing notion of oplax natural transformations between, and tries to narrow the current gap between lax and oplax functors in the library, where the latter has much more formalized API. For maintainability, The code tries to stay as aligned as possible with the code in `CategoryTheory.Bicategory.Naturaltransformations.Oplax`.
---
I followed the book by Johnson and Yau for the definition.
I made @yuma-mizuno and @callesonne authors of the files, as they are the authors of the original code for Oplax functors, which I basically copy-pasted and modified to make it work with lax functors. They should feel free to modify this if they want.
Next thing on the list is to tackle modifications between lax/strong natural transforms of lax transforms, as well as the category instance on lax functors.
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #25565.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/25565* |
t-category-theory |
286/0 |
Mathlib.lean,Mathlib/CategoryTheory/Bicategory/NaturalTransformation/Lax.lean,scripts/noshake.json |
3 |
3 |
['github-actions', 'yuma-mizuno'] |
nobody |
14-73273 14 days ago |
14-73318 14 days ago |
36-31686 36 days |
19668 |
YaelDillies author:YaelDillies |
refactor: define `≤`/`<` on `WithBot`/`WithTop` by induction |
The motivation for this change is that it is really confusing to run `intro r s shouldnthaveintroedthat` on a goal of the form `∀ r s : ℝ≥0∞, r ≤ s` and get the nonsense-looking goal `r = ↑shouldnthaveintroedthat → ∃ b : α, s = ↑b ∧ shouldnthaveintroedthat ≤ b⟩` instead of an error, and similarly when destructing something of the form `∃ r s : ℝ≥0∞, r < s`.
Furthermore, I suspect this improves performance.
---
- [x] depends on: #20317
- [x] depends on: #20318
- [x] depends on: #21274
- [x] depends on: #22109
[](https://gitpod.io/from-referrer/)
|
t-order |
68/51 |
Mathlib/Algebra/Order/Monoid/Unbundled/WithTop.lean,Mathlib/Analysis/Analytic/OfScalars.lean,Mathlib/Analysis/Oscillation.lean,Mathlib/Data/Finset/Lattice/Fold.lean,Mathlib/Data/Finset/Max.lean,Mathlib/LinearAlgebra/Eigenspace/Triangularizable.lean,Mathlib/MeasureTheory/Integral/Lebesgue/Countable.lean,Mathlib/MeasureTheory/Measure/LevyProkhorovMetric.lean,Mathlib/Order/Interval/Basic.lean,Mathlib/Order/Interval/Set/WithBotTop.lean,Mathlib/Order/KrullDimension.lean,Mathlib/Order/WithBot.lean,Mathlib/Probability/Moments/Variance.lean,Mathlib/RingTheory/PowerBasis.lean,Mathlib/Topology/MetricSpace/Holder.lean,Mathlib/Topology/MetricSpace/HolderNorm.lean,MathlibTest/hint.lean |
17 |
20 |
['YaelDillies', 'b-mehta', 'eric-wieser', 'github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'urkud'] |
nobody |
14-69358 14 days ago |
63-73673 2 months ago |
113-66224 113 days |
25743 |
robin-carlier author:robin-carlier |
feat(AlgebraicTopology/SimplexCategory/Augmented): monoidal structure on `AugmentedSimplexCategory` |
We construct a monoidal category structure on `AugmentedSimplexCategory`. The tensor products corresponds to ordinal sum. We characterize morphisms out of a tensor product of object in terms of their precomposition with canonical maps `x ⟶ x ⊗ y` and `y ⟶ x ⊗ y` coming from the fact that the unit is an initial object.
When constructing this structure, we found that making `AugmentedSimplexCategory` an abbrev rather than a `def`
worked better.
---
- [x] depends on: #25742
Future work includes using this monoidal structure and Day convolution to define the join monoidal structure on augmented simplicial sets, and also using this category as a way to encode monoidal and monadic bar constructions.
Happy to discuss the fact that I had to make `AugmentedSimplexCategory` an abbrev, I can revert this but this makes the proofs a bit harder (but, I guess, also less abusing some of defeqs?).
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #22768.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/22768* |
t-topology
t-category-theory
|
523/111 |
Mathlib.lean,Mathlib/AlgebraicTopology/SimplexCategory/Augmented.lean,Mathlib/AlgebraicTopology/SimplexCategory/Augmented/Basic.lean,Mathlib/AlgebraicTopology/SimplexCategory/Augmented/Monoidal.lean,Mathlib/AlgebraicTopology/SimplexCategory/Basic.lean |
5 |
4 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'robin-carlier'] |
nobody |
14-59756 14 days ago |
14-74407 14 days ago |
34-25879 34 days |
26783 |
matthewjasper author:matthewjasper |
feat(RingTheory/Flat): Add theorems relating Submodule.torsion and Module.Flat |
Co-authored-by: Kevin Buzzard
---
This PR continues the work from #25334.
[](https://gitpod.io/from-referrer/)
|
FLT
new-contributor
t-algebra
label:t-algebra$ |
202/0 |
Mathlib.lean,Mathlib/Algebra/Algebra/Bilinear.lean,Mathlib/Algebra/Module/LocalizedModule/Basic.lean,Mathlib/RingTheory/Flat/TorsionFree.lean,Mathlib/RingTheory/Ideal/IsPrincipal.lean |
5 |
1 |
['github-actions'] |
nobody |
14-57720 14 days ago |
14-57746 14 days ago |
14-57775 14 days |
25861 |
robin-carlier author:robin-carlier |
feat(CategoryTheory/Monoidal/Action): action of opposite categories |
Given a monoidal category `C` and a category `D`, we show that left (resp. right) `C`-actions on `D` induce left (resp. right) `Cᵒᵖ`-actions on `Dᵒᵖ`. Conversely, we show that left/right actions of `Cᵒᵖ` on `Dᵒᵖ` induce left/right actions of `C` on `D`.
---
- [ ] depends on: #25860
[](https://gitpod.io/from-referrer/)
|
t-category-theory |
272/0 |
Mathlib/CategoryTheory/Monoidal/Action/Opposites.lean |
1 |
4 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
14-50704 14 days ago |
14-50727 14 days ago |
14-55004 14 days |
25875 |
robin-carlier author:robin-carlier |
feat(CategoryTheory/Monoidal/Action): actions as monoidal functors to endofunctors |
Given a monoidal category `C` and a category `D`, we show that left actions of `C` on `D` correspond to monoidal functors `C ⥤ (D ⥤ D)ᴹᵒᵖ` by showing that the composition of `curriedAction C D` with `mopFunctor` is monoidal, and in the other direction by defining an action of `C` on `D` out of the data of such a monoidal functor.
Similarly, we show that monoidal functors `C ⥤ (D ⥤ D)` correspond to right actions of `C` on `D`.
We use this to define the "evaluation" right action of `(C ⥤ C)` (with the composition monoidal structure) on `C` as the action corresponding to the identity functor `(C ⥤ C) ⥤ (C ⥤ C)`.
---
- [x] depends on: #25840
- [x] depends on: #25766
[](https://gitpod.io/from-referrer/)
|
t-category-theory |
222/3 |
Mathlib.lean,Mathlib/CategoryTheory/Monoidal/Action/Basic.lean,Mathlib/CategoryTheory/Monoidal/Action/End.lean,Mathlib/CategoryTheory/Monoidal/Opposite.lean |
4 |
4 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
14-50543 14 days ago |
14-50561 14 days ago |
27-15044 27 days |
25267 |
YaelDillies author:YaelDillies |
feat: `counit (antipode a) = counit a` |
and unsimp `sum_antipode_mul_eq_algebraMap_counit`/`sum_mul_antipode_eq_algebraMap_counit` since they are annoying lemmas to fight against.
From Toric
Co-authored-by: Patrick Massot
---
[](https://gitpod.io/from-referrer/)
|
toric
t-algebra
label:t-algebra$ |
51/18 |
Mathlib/RingTheory/Coalgebra/Basic.lean,Mathlib/RingTheory/HopfAlgebra/Basic.lean,Mathlib/RingTheory/HopfAlgebra/MonoidAlgebra.lean |
3 |
10 |
['YaelDillies', 'erdOne', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant'] |
nobody |
14-50423 14 days ago |
14-78187 14 days ago |
52-31360 52 days |
25182 |
YaelDillies author:YaelDillies |
feat: `(M →* N₁) ≃* (M →* N₂)` if `N₁ ≃* N₂` |
From Toric
---
[](https://gitpod.io/from-referrer/)
|
toric
t-algebra
label:t-algebra$ |
65/12 |
Mathlib/Algebra/Category/Grp/ForgetCorepresentable.lean,Mathlib/Algebra/Category/Grp/LargeColimits.lean,Mathlib/Algebra/Category/MonCat/ForgetCorepresentable.lean,Mathlib/Algebra/Group/Equiv/Basic.lean,Mathlib/GroupTheory/FiniteAbelian/Duality.lean |
5 |
12 |
['YaelDillies', 'b-mehta', 'eric-wieser', 'github-actions'] |
eric-wieser assignee:eric-wieser |
14-45828 14 days ago |
14-55886 14 days ago |
55-59540 55 days |
26653 |
Hagb author:Hagb |
feat(RingTheory/Finiteness/Defs): span of a set is finitely generated iff generated by a finite subset |
---
This PR continues the work from #24651.
Original PR: #24651.
[](https://gitpod.io/from-referrer/)
|
|
14/0 |
Mathlib/RingTheory/Finiteness/Defs.lean |
1 |
1 |
['github-actions'] |
nobody |
14-44028 14 days ago |
14-44053 14 days ago |
16-76252 16 days |
22151 |
alreadydone author:alreadydone |
feat(RingTheory): a semiprimary ring is Noetherian/Artinian iff its Jacobson radical is fg |
A key fact used is `Module.FG.smul`: if `I` is a two-sided ideal of `R` that is f.g. as a left ideal and `N` is a f.g. `R`-module, then `I • M` is also a f.g. `R`-module.
Many lemmas about coprimality of ideals are also generalized to the noncommutative, two-sided setting.
---
- [x] depends on: #21904
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
217/157 |
Mathlib/Algebra/Algebra/Operations.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Affine/Point.lean,Mathlib/NumberTheory/RamificationInertia/Basic.lean,Mathlib/RingTheory/Extension/Basic.lean,Mathlib/RingTheory/Finiteness/Basic.lean,Mathlib/RingTheory/Finiteness/Ideal.lean,Mathlib/RingTheory/HopkinsLevitzki.lean,Mathlib/RingTheory/Ideal/Maps.lean,Mathlib/RingTheory/Ideal/Operations.lean |
9 |
8 |
['alreadydone', 'github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
14-27635 14 days ago |
14-30817 14 days ago |
136-67620 136 days |
25491 |
tannerduve author:tannerduve |
feat(Control/Monad/Free): define free monad, prove it lawful, and implement standard effects |
This PR introduces the `Free` monad. This implementation uses the "freer monad" approach as the traditional free monad (eg from [Haskell](https://hackage.haskell.org/package/free-5.2/docs/Control-Monad-Free.html)) is not safely definable in Lean due to termination checking (it's not strictly positive).
The main contributions are:
* Definition of the `Free` monad as an inductive type which generates a monad given any type constructor `F : Type -> Type`.
* Functor and Monad instances for `Free F`, along with proofs of the `LawfulFunctor` and `LawfulMonad` laws.
* Canonical instances of `Free` with standard effect signatures:
* `FreeState s` for stateful computations, defined via a `StateF s` functor with `get` and `put` operations.
* `FreeWriter w` for logging computations, defined via a `WriterF w` functor with a `tell` operation.
* `FreeCont r` for continuation-passing computations, using the CPS functor `(α → r) → r`.
In this construction, computations are represented as **trees of effects**. Each node (`liftBind`)
represents a request to perform an effect, accompanied by a continuation specifying how the
computation proceeds after the effect. The leaves (`pure`) represent completed computations with
final results.
A key insight is that `FreeM F` satisfies the **universal property of free monads**: for any monad
`M` and effect handler `f : F → M`, there exists a unique way to interpret `FreeM F` computations
in `M` that respects the effect semantics given by `f`. This unique interpreter is `liftM f`, which
acts as the canonical **fold** for free monads.
To execute or interpret these computations, we provide two approaches:
1. **Hand-written interpreters** (`FreeState.run`, `FreeWriter.run`, `FreeCont.run`) that directly
pattern-match on the tree structure
2. **Canonical interpreters** (`FreeState.toStateM`, `FreeWriter.toWriteT`, `FreeCont.toContT`) derived from
the universal property via `liftM`
And then prove that these approaches are equivalent
---
This PR adds new files and definitions; no breaking changes.
**Tags:** free monad, freer monad, effect systems, state monad, writer monad, continuation monad, operational semantics, verified interpreters
|
t-data
maintainer-merge
|
696/0 |
Mathlib.lean,Mathlib/Control/Monad/Free.lean,Mathlib/Control/Monad/Free/Effects.lean,MathlibTest/freemonad.lean,docs/references.bib |
5 |
145 |
['YaelDillies', 'copilot-pull-request-reviewer', 'eric-wieser', 'github-actions', 'plp127', 'quangvdao', 'tannerduve'] |
nobody |
14-14073 14 days ago |
32-47487 1 month ago |
42-66569 42 days |
26806 |
jcommelin author:jcommelin |
chore: add defeq test for grind rings |
This PR adds a defeq test for multiple paths that convert rings in Mathlib's algebraic hierarchy to abelian groups in grind's hierarchy.
This defeq test used to fail before `leanprover/lean4:v4.22.0-rc3`.
---
[](https://gitpod.io/from-referrer/)
|
|
4/0 |
MathlibTest/grind/ring.lean |
1 |
1 |
['github-actions'] |
nobody |
13-81548 13 days ago |
13-85845 13 days ago |
13-85827 13 days |
26547 |
robin-carlier author:robin-carlier |
feat(CategoryTheory/Limits/Shapes/Pullback/Categorical/CatCospanTransform): more lemmas about isomorphisms of `CatCospanTransform` |
We construct ways to extract left, right or base components of ismorphisms of `CatCospanTransform`, as well as various `IsIso` instances, and lemmas allowing to compute the left, right or base component of the inverse of a `CatCospanTransformMorphism` that has an `IsIso` instance.
---
- [x] depends on: #26412
[](https://gitpod.io/from-referrer/)
|
t-category-theory |
70/0 |
Mathlib/CategoryTheory/Limits/Shapes/Pullback/Categorical/CatCospanTransform.lean |
1 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
13-74463 13 days ago |
14-67632 14 days ago |
14-70679 14 days |
24998 |
YaelDillies author:YaelDillies |
chore(Algebra/Notation): separate very basic lemmas about `Set.indicator` and `Pi.single` |
The very basic lemmas go under `Algebra.Notation` and do not import `Monoid`.
This is useful to disentangle `Finsupp` results downstream.
---
- [x] depends on: #25040
[](https://gitpod.io/from-referrer/)
|
file-removed |
719/640 |
Mathlib.lean,Mathlib/Algebra/BigOperators/Finprod.lean,Mathlib/Algebra/BigOperators/Group/Finset/Lemmas.lean,Mathlib/Algebra/BigOperators/GroupWithZero/Finset.lean,Mathlib/Algebra/BigOperators/Pi.lean,Mathlib/Algebra/Divisibility/Prod.lean,Mathlib/Algebra/Group/End.lean,Mathlib/Algebra/Group/Equiv/TypeTags.lean,Mathlib/Algebra/Group/Fin/Tuple.lean,Mathlib/Algebra/Group/Finsupp.lean,Mathlib/Algebra/Group/Hom/Defs.lean,Mathlib/Algebra/Group/Indicator.lean,Mathlib/Algebra/Group/Nat/Hom.lean,Mathlib/Algebra/Group/NatPowAssoc.lean,Mathlib/Algebra/Group/Pi/Basic.lean,Mathlib/Algebra/Group/Pointwise/Set/Scalar.lean,Mathlib/Algebra/Group/Prod.lean,Mathlib/Algebra/Group/Support.lean,Mathlib/Algebra/Group/TypeTags/Basic.lean,Mathlib/Algebra/GroupWithZero/Action/Defs.lean,Mathlib/Algebra/GroupWithZero/Indicator.lean,Mathlib/Algebra/Homology/Additive.lean,Mathlib/Algebra/Module/Basic.lean,Mathlib/Algebra/Notation/FiniteSupport.lean,Mathlib/Algebra/Notation/Indicator.lean,Mathlib/Algebra/Notation/Pi/Basic.lean,Mathlib/Algebra/Notation/Pi/Defs.lean,Mathlib/Algebra/Notation/Support.lean,Mathlib/Algebra/Order/Field/Pi.lean,Mathlib/Algebra/Order/Group/Unbundled/Abs.lean,Mathlib/Algebra/Order/GroupWithZero/Unbundled/Basic.lean,Mathlib/Algebra/Order/Sub/Prod.lean,Mathlib/Algebra/Order/Sum.lean,Mathlib/Algebra/Ring/CharZero.lean,Mathlib/Algebra/Ring/Hom/Defs.lean,Mathlib/CategoryTheory/Limits/Shapes/ZeroMorphisms.lean,Mathlib/Combinatorics/Additive/Dissociation.lean,Mathlib/Combinatorics/SimpleGraph/Bipartite.lean,Mathlib/Data/Finsupp/Basic.lean,Mathlib/Data/Finsupp/Defs.lean,Mathlib/Data/Finsupp/Single.lean,Mathlib/Data/Int/CharZero.lean,Mathlib/Data/Set/Pointwise/Support.lean,Mathlib/GroupTheory/FreeGroup/Basic.lean,Mathlib/MeasureTheory/MeasurableSpace/Basic.lean,Mathlib/Order/Filter/Basic.lean,Mathlib/Order/Filter/EventuallyConst.lean,Mathlib/Order/Interval/Set/Pi.lean,Mathlib/RingTheory/HahnSeries/Addition.lean,Mathlib/RingTheory/HahnSeries/Basic.lean,Mathlib/Topology/Algebra/Indicator.lean,Mathlib/Topology/IndicatorConstPointwise.lean,Mathlib/Topology/LocallyConstant/Basic.lean,Mathlib/Topology/LocallyFinsupp.lean,Mathlib/Topology/Separation/Basic.lean,Mathlib/Topology/Separation/DisjointCover.lean |
56 |
13 |
['YaelDillies', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
13-70554 13 days ago |
13-70600 13 days ago |
54-20950 54 days |
24719 |
madvorak author:madvorak |
feat(LinearAlgebra/Matrix/NonsingularInverse): inverting `Matrix` inverts its `LinearEquiv` |
---
Discussion:
https://leanprover.zulipchat.com/#narrow/channel/144837-PR-reviews/topic/.2324719.20cannot.20find.20home/with/517142655
|
t-algebra label:t-algebra$ |
10/0 |
Mathlib/LinearAlgebra/Matrix/NonsingularInverse.lean |
1 |
15 |
['eric-wieser', 'github-actions', 'madvorak'] |
nobody |
13-69158 13 days ago |
69-54347 2 months ago |
71-4173 71 days |
26746 |
alreadydone author:alreadydone |
feat(RingTheory): integral extensions of comm. rings are local homs |
migrated from #23684
---
The import increase only affects one file so I hope it's okay.
[](https://gitpod.io/from-referrer/) |
large-import |
59/66 |
Mathlib/Algebra/Field/Equiv.lean,Mathlib/Algebra/Group/Invertible/Basic.lean,Mathlib/Algebra/GroupWithZero/Units/Basic.lean,Mathlib/AlgebraicGeometry/Morphisms/Proper.lean,Mathlib/FieldTheory/LinearDisjoint.lean,Mathlib/LinearAlgebra/Dimension/Localization.lean,Mathlib/NumberTheory/RamificationInertia/Unramified.lean,Mathlib/RingTheory/Artinian/Ring.lean,Mathlib/RingTheory/Ideal/Int.lean,Mathlib/RingTheory/IntegralClosure/Algebra/Defs.lean,Mathlib/RingTheory/IntegralClosure/IsIntegralClosure/Basic.lean,Mathlib/RingTheory/LinearDisjoint.lean,Mathlib/RingTheory/Localization/FractionRing.lean,Mathlib/RingTheory/Localization/Integral.lean,Mathlib/RingTheory/SimpleRing/Field.lean |
15 |
7 |
['alreadydone', 'github-actions', 'leanprover-bot', 'mariainesdff'] |
mariainesdff assignee:mariainesdff |
13-66625 13 days ago |
13-66625 13 days ago |
15-50189 15 days |
26608 |
vihdzp author:vihdzp |
feat(SetTheory/Cardinal/Aleph): `o.card ≤ ℵ_ o` and variants |
---
[](https://gitpod.io/from-referrer/)
|
t-set-theory |
24/0 |
Mathlib/SetTheory/Cardinal/Aleph.lean |
1 |
2 |
['github-actions', 'kckennylau'] |
nobody |
13-59751 13 days ago |
18-6988 18 days ago |
18-7735 18 days |
26607 |
vihdzp author:vihdzp |
feat(SetTheory/Cardinal/Aleph): characterization of initial successor ordinals |
---
[](https://gitpod.io/from-referrer/)
|
t-set-theory |
5/0 |
Mathlib/SetTheory/Cardinal/Aleph.lean |
1 |
5 |
['github-actions', 'kckennylau', 'vihdzp'] |
nobody |
13-49616 13 days ago |
18-7772 18 days ago |
18-7817 18 days |
26770 |
Jun2M author:Jun2M |
feat(Combinatorics/Graph) : subgraph relations and operations on `Graph` |
This PR creates a new file `Combinatorics/Graph/Subgraph.lean`. In it, the PR introduces a partial order on graphs by subgraph relation, defines relations `IsInducedSubgraph`, `IsSpanningSubgraph` and `IsClosedSubgraph`. Further, it introduce operations `EdgeRestrict`, `EdgeDelete`, `induce` and `VertexDelete`.
Co-authored-by: Peter Nelson
---
[](https://gitpod.io/from-referrer/)
|
t-combinatorics |
703/0 |
Mathlib.lean,Mathlib/Combinatorics/Graph/Subgraph.lean |
2 |
1 |
['github-actions'] |
nobody |
13-34347 13 days ago |
15-23161 15 days ago |
15-23205 15 days |
26829 |
pechersky author:pechersky |
feat(RingTheory/Valuation): Valuation.leAddSubgroup and ideal/submodule versions of ltAddSubgroup |
Extracted from #25450 without changing how Valued works
---
[](https://gitpod.io/from-referrer/)
@faenuccio hopefully this bypasses any wait on #14752 because I am not changing Valued files. |
t-algebra label:t-algebra$ |
177/0 |
Mathlib/RingTheory/Valuation/Basic.lean,Mathlib/RingTheory/Valuation/Integers.lean |
2 |
1 |
['github-actions'] |
nobody |
13-20456 13 days ago |
13-25974 13 days ago |
13-26029 13 days |
26617 |
vihdzp author:vihdzp |
feat(Data/Sum/Order): `toLex` as a `RelIso` |
As [requested](https://github.com/leanprover-community/mathlib4/pull/20409#discussion_r1903319844) by @eric-wieser in #20409.
---
[](https://gitpod.io/from-referrer/)
|
t-data
t-order
|
30/0 |
Mathlib/Data/Sum/Order.lean |
1 |
4 |
['eric-wieser', 'github-actions', 'kckennylau', 'vihdzp'] |
nobody |
13-14833 13 days ago |
18-1181 18 days ago |
18-1444 18 days |
26723 |
chrisflav author:chrisflav |
feat(AlgebraicGeometry): source-local closure of a morphism property |
As a special case, we define local isomorphisms as the source local closure of open immersions.
---
[](https://gitpod.io/from-referrer/)
|
t-algebraic-geometry |
170/0 |
Mathlib.lean,Mathlib/AlgebraicGeometry/Morphisms/LocalClosure.lean,Mathlib/AlgebraicGeometry/Morphisms/LocalIso.lean |
3 |
6 |
['chrisflav', 'github-actions', 'joelriou'] |
nobody |
13-14809 13 days ago |
13-14809 13 days ago |
15-53142 15 days |
26822 |
jsm28 author:jsm28 |
feat(LinearAlgebra/AffineSpace): affine combinations and spans of images |
Add two lemmas about affine combinations and the spans of points in a subset of an indexed family.
```lean
/-- A point in the `affineSpan` of a subset of an indexed family is an
`affineCombination` with sum of weights 1, using only points in the given subset. -/
lemma eq_affineCombination_of_mem_affineSpan_image {p₁ : P} {p : ι → P} {s : Set ι}
(h : p₁ ∈ affineSpan k (p '' s)) :
∃ (fs : Finset ι) (w : ι → k), ↑fs ⊆ s ∧ ∑ i ∈ fs, w i = 1 ∧
p₁ = fs.affineCombination k p w := by
```
```lean
/-- If an affine combination of affinely independent points lies in the affine span of a subset
of those points, all weights outside that subset are zero. -/
lemma AffineIndependent.eq_zero_of_affineCombination_mem_affineSpan {p : ι → P}
(ha : AffineIndependent k p) {fs : Finset ι} {w : ι → k} (hw : ∑ i ∈ fs, w i = 1) {s : Set ι}
(hm : fs.affineCombination k p w ∈ affineSpan k (p '' s)) {i : ι} (hifs : i ∈ fs)
(his : i ∉ s) : w i = 0 := by
```
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
27/0 |
Mathlib/LinearAlgebra/AffineSpace/Combination.lean,Mathlib/LinearAlgebra/AffineSpace/Independent.lean |
2 |
1 |
['github-actions'] |
nobody |
13-14134 13 days ago |
13-37774 13 days ago |
13-37757 13 days |
26833 |
pechersky author:pechersky |
feat(ValuativeRel): MulArchimedean (ValueGroupWithZero R) when IsRankLeOne |
with a proof_wanted for the reverse implication
---
[](https://gitpod.io/from-referrer/)
|
t-order
t-algebra
t-number-theory
label:t-algebra$ |
12/0 |
Mathlib/RingTheory/Valuation/ValuativeRel.lean |
1 |
1 |
['github-actions'] |
nobody |
13-306 13 days ago |
13-358 13 days ago |
13-357 13 days |
26785 |
TOMILO87 author:TOMILO87 |
feat: beta distribution |
Add the Beta distribution to the probability distributions in mathlib4.
This implementation includes:
- Definition of the Beta function over the reals
- The probability density function (PDF) of the Beta distribution
- Proof that the PDF integrates to 1
- The corresponding `Measure` and CDF
- Lemmas about measurability, positivity, and integrability
The Beta distribution is a family of continuous probability distributions defined on the interval [0, 1], parametrized by two positive shape parameters, `α` and `β`, that control the shape of the distribution.
This follows the general structure of other distributions in mathlib, such as the Gamma distribution.
---
This is a clean version of the PR originally opened as [#25608](https://github.com/leanprover-community/mathlib4/pull/25608) and temporarily migrated in [#26325](https://github.com/leanprover-community/mathlib4/pull/26325).
It includes:
- `456da1c`: Initial version of the distribution
- `c047aee`: Address review comments from @EtienneC30
- `f165c79`: Remove `ae` condition from `lintegral_betaPDF_eq`
- `7875f47`: Lint fix for unused simp args
This PR is rebased onto `master` and follows the fork-based workflow.
Thanks for your helpful comments earlier!
|
new-contributor
t-measure-probability
|
285/0 |
Mathlib.lean,Mathlib/Analysis/SpecialFunctions/Gamma/Beta.lean,Mathlib/Probability/Distributions/Beta.lean |
3 |
1 |
['github-actions'] |
nobody |
12-73869 12 days ago |
12-73869 12 days ago |
14-50725 14 days |
26841 |
xroblot author:xroblot |
feat(FieldTheory/IsGalois): map induced by the restriction to a subfield |
For `E/L` a field extension and `K` a subfield of `E`, we define the map `(E ≃ₐ[L] E) →* (K ≃ₐ[F] K)` induced by the restriction to `K` (with `F` a subfield of `K` and `L` such that `K/F` is normal) and study when it is injective and surjective.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
63/0 |
Mathlib/FieldTheory/Galois/Basic.lean |
1 |
1 |
['github-actions'] |
nobody |
12-72749 12 days ago |
12-73021 12 days ago |
12-73068 12 days |
26845 |
kbuzzard author:kbuzzard |
chore: rename ValuativeTopology to IsValuativeTopology |
---
[](https://gitpod.io/from-referrer/)
It's a Prop but it involves topology so we have two conflicting naming conventions, namely the topologists "`CompactSpace` is a perfectly fine name for a Prop and anyway we got used to it now" convention, and everyone else's `Is` convention. We're not used to this yet though so let's fix it.
|
t-algebra label:t-algebra$ |
2/2 |
Mathlib/RingTheory/Valuation/ValuativeRel.lean |
1 |
1 |
['github-actions'] |
nobody |
12-70194 12 days ago |
12-70202 12 days ago |
12-70248 12 days |
26271 |
Raph-DG author:Raph-DG |
feat(AlgebraicGeometry): Simple lemma about existence of affine neighbourhoods |
In this PR we make a simple lemma saying there exists an affine open around any point in a scheme. This already exists in the language of open immersions, this just makes the construction of the affine open subset more convenient.
---
[](https://gitpod.io/from-referrer/)
|
t-algebraic-geometry |
6/0 |
Mathlib/AlgebraicGeometry/AffineScheme.lean |
1 |
1 |
['github-actions'] |
nobody |
12-63974 12 days ago |
27-46937 27 days ago |
27-46981 27 days |
25776 |
Parcly-Taxel author:Parcly-Taxel |
chore: deprime `induction` in `Analysis` |
I think this is very marginally dependent on #25770. |
tech debt
t-analysis
|
256/208 |
Mathlib/Analysis/Analytic/Composition.lean,Mathlib/Analysis/Analytic/Constructions.lean,Mathlib/Analysis/Analytic/Inverse.lean,Mathlib/Analysis/BoxIntegral/Basic.lean,Mathlib/Analysis/BoxIntegral/Box/SubboxInduction.lean,Mathlib/Analysis/BoxIntegral/Partition/Additive.lean,Mathlib/Analysis/BoxIntegral/Partition/Split.lean,Mathlib/Analysis/CStarAlgebra/Basic.lean,Mathlib/Analysis/CStarAlgebra/Multiplier.lean,Mathlib/Analysis/Calculus/ContDiff/Basic.lean,Mathlib/Analysis/Calculus/ContDiff/Bounds.lean,Mathlib/Analysis/Calculus/ContDiff/FTaylorSeries.lean,Mathlib/Analysis/Calculus/ContDiff/Operations.lean,Mathlib/Analysis/Calculus/Deriv/ZPow.lean,Mathlib/Analysis/Calculus/InverseFunctionTheorem/ApproximatesLinearOn.lean,Mathlib/Analysis/Calculus/IteratedDeriv/Lemmas.lean,Mathlib/Analysis/Calculus/SmoothSeries.lean,Mathlib/Analysis/Convex/Combination.lean,Mathlib/Analysis/Convex/Radon.lean,Mathlib/Analysis/InnerProductSpace/Projection.lean,Mathlib/Analysis/Normed/Algebra/Exponential.lean,Mathlib/Analysis/NormedSpace/Multilinear/Basic.lean,Mathlib/Analysis/Seminorm.lean,Mathlib/Analysis/SpecialFunctions/Complex/Arg.lean,Mathlib/Analysis/SpecialFunctions/Complex/Circle.lean,Mathlib/Analysis/SpecialFunctions/Gamma/Basic.lean,Mathlib/Analysis/SpecialFunctions/Gamma/Beta.lean,Mathlib/Analysis/SpecialFunctions/Gamma/BohrMollerup.lean,Mathlib/Analysis/SpecialFunctions/Gamma/Deriv.lean,Mathlib/Analysis/SpecialFunctions/Integrals/Basic.lean,Mathlib/Analysis/SpecialFunctions/Log/Basic.lean,Mathlib/Analysis/SpecialFunctions/Pow/Deriv.lean,Mathlib/Analysis/SpecialFunctions/Pow/NNReal.lean,Mathlib/Analysis/SpecialFunctions/Pow/Real.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/EulerSineProd.lean |
35 |
3 |
['Parcly-Taxel', 'github-actions', 'leanprover-community-bot-assistant', 'madvorak'] |
nobody |
12-62913 12 days ago |
13-10485 13 days ago |
35-77061 35 days |
26765 |
KiringYJ author:KiringYJ |
feat(MeasureTheory/PiSystem): add π-λ theorem and SetLike instance |
Add two small features to `MeasureTheory/PiSystem`:
1. SetLike instance
`instance : SetLike (DynkinSystem α) (Set α)`
This lets us write `s ⊆ d` and `t ∈ d` for a DynkinSystem `d`, matching usual mathlib style.
2. `DynkinSystem.pi_lambda` lemma
Classical π‑λ theorem: if a π‑system `s` is contained in a Dynkin system `d`, every set measurable for `σ(s)` is also in `d`.
Currently, mathlib exposes this result only indirectly (e.g. via `generateFrom_eq`). Although logically equivalent, it is not obvious at first glance that those lemmas are the π‑λ theorem. The new lemma states the result in its familiar textbook form, so users can recognise and cite it immediately.
Both pieces are under 10 lines, term‑mode only, and do not modify existing APIs.
No breaking changes.
No dependencies.
|
new-contributor
t-measure-probability
easy
|
13/0 |
Mathlib/MeasureTheory/PiSystem.lean |
1 |
10 |
['KiringYJ', 'github-actions', 'ocfnash'] |
nobody |
12-51867 12 days ago |
12-75120 12 days ago |
15-35575 15 days |
26219 |
Thmoas-Guan author:Thmoas-Guan |
feat(RingTheory/KrullDimension): Krull Dimension of quotient regular sequence |
We show that if M is a finite module over a Noetherian local ring R, [r₁, …, rₙ] is an M-sequence, then dim M⧸(r₁, …, rₙ)M + n = dim M.
Co-authored-by: Yongle Hu @mbkybky
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
220/30 |
Mathlib.lean,Mathlib/Algebra/Module/Submodule/Lattice.lean,Mathlib/LinearAlgebra/Quotient/Basic.lean,Mathlib/RingTheory/Ideal/MinimalPrime/Localization.lean,Mathlib/RingTheory/KrullDimension/Module.lean,Mathlib/RingTheory/KrullDimension/Regular.lean,Mathlib/RingTheory/Nakayama.lean,Mathlib/RingTheory/Spectrum/Prime/LTSeries.lean,Mathlib/RingTheory/Support.lean |
9 |
3 |
['Thmoas-Guan', 'github-actions', 'leanprover-community-bot-assistant'] |
nobody |
12-48927 12 days ago |
13-2907 13 days ago |
27-62518 27 days |
26790 |
FlAmmmmING author:FlAmmmmING |
feat(Combinatorics/Enumerative/Bell.lean): define standard Bell number |
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-combinatorics
|
38/1 |
Mathlib/Combinatorics/Enumerative/Bell.lean |
1 |
11 |
['AntoineChambert-Loir', 'FlAmmmmING', 'eric-wieser', 'github-actions', 'kckennylau', 'madvorak'] |
nobody |
12-46834 12 days ago |
14-43496 14 days ago |
14-43542 14 days |
26844 |
kebekus author:kebekus |
feat: establish examples of harmonic functions |
If `f : ℂ → F` is complex-differentiable, then show that `f` is harmonic. If `F = ℂ`, then so is its real part, imaginary part, and complex conjugate. If `f` has no zero, then `log ‖f‖` is harmonic.
This material is used in [Project VD](https://github.com/kebekus/ProjectVD), which aims to formalize Value Distribution Theory for meromorphic functions on the complex plane. It is one of the ingredients in the proof of Jensen's Formula in complex analysis.
---
[](https://gitpod.io/from-referrer/)
|
t-analysis |
129/0 |
Mathlib.lean,Mathlib/Analysis/Complex/Basic.lean,Mathlib/Analysis/InnerProductSpace/Harmonic/Constructions.lean |
3 |
9 |
['github-actions', 'grunweg', 'kebekus'] |
nobody |
12-44395 12 days ago |
12-70282 12 days ago |
12-70330 12 days |
26835 |
Vtec234 author:Vtec234 |
feat(Tactic): dependent rewriting ct'd |
Add dependent rewrite tactics `rw!` and `rewrite!`.
These operate by inserting casts in front of terms that would otherwise become type-incorrect after the rewrite.
In the default mode, only proof terms are casted, so that (by proof irrelevance) no observable complexity is added.
In the most liberal mode, the tactics never encounter the 'motive is not type correct' error,
but may add casts that make the goal or other term very complex.
Co-authored-by: Aaron Liu
---
Continued from #23930.
This has been discussed on Zulip [here](https://leanprover.zulipchat.com/#narrow/channel/239415-metaprogramming-.2F-tactics/topic/dependent.20rewrite.20tactic/with/504228516). See the included test file for example rewrites that this tactic can do.
[](https://gitpod.io/from-referrer/)
|
t-meta |
764/0 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/DepRewrite.lean,MathlibTest/depRewrite.lean |
4 |
5 |
['Vtec234', 'github-actions', 'kmill', 'plp127'] |
nobody |
12-40369 12 days ago |
12-81934 12 days ago |
12-81985 12 days |
25856 |
MichaelStollBayreuth author:MichaelStollBayreuth |
perf(Data.Real.Sqrt): make Real.sqrt irreducible |
We try to see what happens if we make Real.sqrt irreducible.
There are cases where this makes unification very significantly faster, compare [#mathlib4 > Coercion triggers timeout @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Coercion.20triggers.20timeout/near/517177117).
(Migrated manually from #24752)
---
[](https://gitpod.io/from-referrer/)
|
migrated-from-branch
t-data
|
1/0 |
Mathlib/Data/Real/Sqrt.lean |
1 |
1 |
['github-actions'] |
nobody |
12-39125 12 days ago |
35-56474 1 month ago |
35-60178 35 days |
26158 |
upobir author:upobir |
feat(NumberTheory/Divisors): add int divisors |
This PR continues the work from #25209.
Original PR: https://github.com/leanprover-community/mathlib4/pull/25209 |
t-number-theory |
101/4 |
Mathlib/NumberTheory/Divisors.lean |
1 |
34 |
['MichaelStollBayreuth', 'github-actions', 'upobir'] |
nobody |
12-30507 12 days ago |
30-51359 1 month ago |
30-51402 30 days |
26693 |
euprunin author:euprunin |
chore: golf Computability/ using `grind` |
|
t-computability |
5/24 |
Mathlib/Computability/Language.lean,Mathlib/Computability/Partrec.lean,Mathlib/Computability/PostTuringMachine.lean,Mathlib/Computability/Primrec.lean,Mathlib/Computability/RegularExpressions.lean |
5 |
4 |
['github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot'] |
nobody |
12-23845 12 days ago |
12-23845 12 days ago |
16-36389 16 days |
26882 |
DavidLedvinka author:DavidLedvinka |
feat(Analysis): Additional `AsymptoticEquivalent` API |
Add four new theorems about asymptotic equivalence. These are used in the Brownian Motion project.
|
large-import
t-analysis
|
36/1 |
Mathlib/Analysis/Asymptotics/AsymptoticEquivalent.lean,Mathlib/Analysis/Asymptotics/SpecificAsymptotics.lean |
2 |
1 |
['github-actions'] |
nobody |
12-22575 12 days ago |
12-28974 12 days ago |
12-29026 12 days |
26689 |
euprunin author:euprunin |
chore: golf Combinatorics/ using `grind` |
|
t-combinatorics |
10/53 |
Mathlib/Combinatorics/Enumerative/Composition.lean,Mathlib/Combinatorics/Enumerative/DyckWord.lean,Mathlib/Combinatorics/Hall/Finite.lean,Mathlib/Combinatorics/SimpleGraph/Connectivity/WalkCounting.lean,Mathlib/Combinatorics/SimpleGraph/Paths.lean,Mathlib/Combinatorics/SimpleGraph/Subgraph.lean,Mathlib/Combinatorics/SimpleGraph/Trails.lean,Mathlib/Combinatorics/SimpleGraph/Triangle/Counting.lean |
8 |
8 |
['bryangingechen', 'github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'leanprover-community-mathlib4-bot'] |
nobody |
12-17753 12 days ago |
12-17753 12 days ago |
16-34596 16 days |
26857 |
Thmoas-Guan author:Thmoas-Guan |
feat(Algebra): define associated graded structure for abelian group |
In this PR we define the associated graded structure for abelian group when given a filtration and only give some basic lemmas about it.
Further results would be given in #26858
---
[](https://gitpod.io/from-referrer/)
migrated from #22631
|
t-algebra label:t-algebra$ |
154/0 |
Mathlib.lean,Mathlib/RingTheory/FilteredAlgebra/AssociatedGraded.lean |
2 |
1 |
['github-actions'] |
nobody |
11-66008 11 days ago |
12-51849 12 days ago |
12-51894 12 days |
26885 |
pechersky author:pechersky |
feat(Topology/ValuativeRel): ValuativeTopology 𝒪[K] |
and even when not a field, `ValuativeRel 𝒪[K]`
This is an example of something achievable with the new declarations that wasn't possible with Valued
Such that we can discuss the valuations on the subring without always using coercions
But to achieve this, one needs some juggling of the value groups
---
[](https://gitpod.io/from-referrer/)
- [x] depends on: #26834
|
t-algebra
t-topology
t-number-theory
label:t-algebra$ |
82/10 |
Mathlib/RingTheory/Valuation/ValuativeRel.lean,Mathlib/Topology/Algebra/Valued/ValuativeRel.lean |
2 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
11-53414 11 days ago |
11-54346 11 days ago |
0-331 5 minutes |
26210 |
Thmoas-Guan author:Thmoas-Guan |
feat(Algebra): associated primes of localized module |
We proved the `Ass(S^{-1}M)` is equal to the preimage of `Ass(M)` under `Ideal.comap` when over noetherian ring.
From this we proved that every minimal primes over `Module.annihilator R M` is in `Ass(M)` when `M` is finitely generated.
---
[](https://gitpod.io/from-referrer/) |
large-import
t-algebra
label:t-algebra$ |
73/15 |
Mathlib/RingTheory/Ideal/AssociatedPrime/Localization.lean |
1 |
9 |
['Thmoas-Guan', 'github-actions', 'mbkybky'] |
nobody |
11-50849 11 days ago |
11-51958 11 days ago |
21-64210 21 days |
26299 |
adomani author:adomani |
perf: the `commandStart` linter only acts on modified files |
Introduces an `IO.Ref` to allow the `commandStart` linter to only run on files that git considers modified with respect to `master`.
The linter is also active on files that have had some error, as these are likely being modified!
The PR should also mitigate the speed-up that the linter introduced:
[#mathlib4 > A whitespace linter @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/A.20whitespace.20linter/near/525091877)
Assuming that this goes well, a similar mechanism could be applied to several linters that do not need to run on all code, just on the modified code.
Implementation detail: the linter is currently either on or off in "whole" files. It may be also a future development to make this more granular and only run the linter on "modifed commands in modified files", but this is not currently the plan for this modification!
---
[](https://gitpod.io/from-referrer/)
|
t-linter |
48/0 |
Mathlib/Tactic/Linter/CommandStart.lean |
1 |
4 |
['adomani', 'github-actions', 'leanprover-bot'] |
nobody |
11-39259 11 days ago |
26-51958 26 days ago |
26-56590 26 days |
26035 |
fbarroero author:fbarroero |
feat(Analysis/Polynomial/MahlerMeasure): the Mahler measure of a complex polynomial |
We introduce the Mahler measure of a complex polynomial and prove some basic facts.
---
[](https://gitpod.io/from-referrer/)
|
t-analysis |
127/1 |
Mathlib.lean,Mathlib/Analysis/Polynomial/MahlerMeasure.lean,Mathlib/MeasureTheory/Integral/CircleIntegral.lean |
3 |
1 |
['github-actions'] |
nobody |
11-31475 11 days ago |
31-42457 1 month ago |
31-42460 31 days |
26909 |
gasparattila author:gasparattila |
feat(LinearAlgebra/Projectivization/Subspace): correspondence between linear and projective subspaces |
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-algebra
label:t-algebra$ |
51/3 |
Mathlib/LinearAlgebra/Projectivization/Subspace.lean |
1 |
1 |
['github-actions'] |
nobody |
11-29289 11 days ago |
11-29295 11 days ago |
11-29343 11 days |
26300 |
igorkhavkine author:igorkhavkine |
feat(Analysis/Calculus/FDeriv): continuous differentiability from continuous partial derivatives on an open domain in a product space |
If a function `f : E × F → G` is continuously differentiable, then its partial derivatives along `E` and `F` are also continuous. The non-trivial converse implication holds when the partial derivatives are continuous on an open domain, and they can be added together to give the total derivative of `f`. See this [#mathlib4 > Partial derivatives @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Partial.20derivatives/near/520995477) and the containing thread for some discussion. The PR creates a new import (`Mathlib.Analysis.Calculus.FDeriv.Partial`), where other results about partial derivatives could go in the future.
---
*this is the migration of #25304 to the PR-from-fork workflow*
- [x] depends on: #25564
- [x] depends on: #26273
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-analysis
|
365/0 |
Mathlib.lean,Mathlib/Analysis/Calculus/FDeriv/Partial.lean,Mathlib/Analysis/Normed/Operator/BoundedLinearMaps.lean |
3 |
7 |
['YaelDillies', 'agjftucker', 'github-actions', 'igorkhavkine', 'mathlib4-dependent-issues-bot'] |
nobody |
11-20495 11 days ago |
23-72503 23 days ago |
24-58241 24 days |
25774 |
Parcly-Taxel author:Parcly-Taxel |
chore: deprime `induction` in `AlgebraicTopology/CategoryTheory` |
Most replacements that are also in #23676 have been copied over, but some have been optimised further. |
tech debt |
131/122 |
Mathlib/AlgebraicTopology/DoldKan/Decomposition.lean,Mathlib/AlgebraicTopology/DoldKan/Degeneracies.lean,Mathlib/AlgebraicTopology/DoldKan/NCompGamma.lean,Mathlib/AlgebraicTopology/DoldKan/Projections.lean,Mathlib/AlgebraicTopology/SimplexCategory/MorphismProperty.lean,Mathlib/AlgebraicTopology/SimplicialObject/Split.lean,Mathlib/AlgebraicTopology/SimplicialSet/Degenerate.lean,Mathlib/AlgebraicTopology/SimplicialSet/NerveAdjunction.lean,Mathlib/AlgebraicTopology/SimplicialSet/StdSimplex.lean,Mathlib/CategoryTheory/Abelian/GrothendieckCategory/EnoughInjectives.lean,Mathlib/CategoryTheory/Abelian/GrothendieckCategory/Subobject.lean,Mathlib/CategoryTheory/Action/Concrete.lean,Mathlib/CategoryTheory/Action/Monoidal.lean,Mathlib/CategoryTheory/ComposableArrows.lean,Mathlib/CategoryTheory/Extensive.lean,Mathlib/CategoryTheory/Filtered/Basic.lean,Mathlib/CategoryTheory/Galois/Decomposition.lean,Mathlib/CategoryTheory/Galois/EssSurj.lean,Mathlib/CategoryTheory/Limits/Shapes/Equalizers.lean,Mathlib/CategoryTheory/Limits/Shapes/SequentialProduct.lean,Mathlib/CategoryTheory/Limits/VanKampen.lean,Mathlib/CategoryTheory/Quotient.lean,Mathlib/CategoryTheory/Sites/Sheaf.lean,Mathlib/CategoryTheory/Subobject/Basic.lean,Mathlib/CategoryTheory/Subobject/FactorThru.lean,Mathlib/CategoryTheory/Subobject/Lattice.lean,Mathlib/CategoryTheory/Triangulated/TStructure/Basic.lean |
27 |
5 |
['Parcly-Taxel', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'madvorak'] |
nobody |
11-1759 11 days ago |
11-1780 11 days ago |
35-73593 35 days |
22322 |
mariainesdff author:mariainesdff |
feat(RingTheory/DividedPowers/RatAlgebra): add definitions |
In this file we show that, for certain choices of a commutative (semi)ring `A` and an ideal `I` of
`A`, the family of maps `ℕ → A → A` given by `fun n x ↦ x^n/n!` is a divided power structure on `I`.
Co-authored-by: AntoineChambert-Loir
---
- [x] depends on: #22237
- [x] depends on: #22239
- [x] depends on: #22240
- [x] depends on: #24439
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
324/2 |
Mathlib.lean,Mathlib/Data/Nat/Factorial/NatCast.lean,Mathlib/RingTheory/DividedPowers/RatAlgebra.lean |
3 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
10-70084 10 days ago |
10-72219 10 days ago |
18-16516 18 days |
25830 |
ScottCarnahan author:ScottCarnahan |
refactor (RingTheory/HahnSeries/HEval): remove positive order condition from definition |
This PR removes the positive order condition for substitution (or Hahn evaluation) of a Hahn series into a power series. When the order is not positive, the function substitutes zero. We also add short lemmas for substitution into `PowerSeries.X` and `PowerSeries.C`.
---
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #24498.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/24498* |
t-algebra label:t-algebra$ |
34/15 |
Mathlib/RingTheory/HahnSeries/HEval.lean |
1 |
2 |
['github-actions', 'leanprover-community-bot-assistant'] |
nobody |
10-69204 10 days ago |
12-35790 12 days ago |
34-39459 34 days |
26928 |
vihdzp author:vihdzp |
feat(Topology/Order/Basic): lower set in well-order is open |
As well as the other analogous theorems.
---
[](https://gitpod.io/from-referrer/)
|
t-topology |
37/0 |
Mathlib/Order/UpperLower/Basic.lean,Mathlib/Topology/Order/Basic.lean |
2 |
1 |
['github-actions'] |
nobody |
10-62918 10 days ago |
10-65058 10 days ago |
10-65246 10 days |
26204 |
Raph-DG author:Raph-DG |
feat(AlgebraicGeometry): Add global preorder instance for schemes |
In this PR we added a default preorder instance for schemes, defined to be the specialization order as discussed here: https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/dimension.20function.20for.20schemes/near/524997376 for discussion
---
[](https://gitpod.io/from-referrer/)
|
t-algebraic-geometry |
18/0 |
Mathlib/AlgebraicGeometry/AffineSpace.lean,Mathlib/AlgebraicGeometry/Scheme.lean |
2 |
11 |
['Raph-DG', 'erdOne', 'github-actions', 'ocfnash'] |
nobody |
10-56549 10 days ago |
13-36309 13 days ago |
28-69194 28 days |
26934 |
mariainesdff author:mariainesdff |
feat(RingTheory/DedekindDomain/Ideal): add HeightOneSpectrum.ofPrime |
Previously #24036.
Co-authored-by: @Louddy
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
9/0 |
Mathlib/RingTheory/DedekindDomain/Ideal.lean |
1 |
2 |
['github-actions', 'riccardobrasca'] |
riccardobrasca assignee:riccardobrasca |
10-50756 10 days ago |
10-54322 10 days ago |
10-54378 10 days |
26936 |
mariainesdff author:mariainesdff |
feat(RingTheory/DividedPowes/SubDPIdeal): complete lattice and quotients |
We show that sub-dp-ideals of a divided power ideal `I` of a ring `A` form a complete lattice under inclusion.
Given an ideal `J` of `A`, we construct the divided power structure on the ideal `I(A⧸J)` of the quotient, provided that `I ⊓ J` is a sub-dp-ideal of `I`.
Co-authored-by: @AntoineChambert-Loir
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebra
label:t-algebra$ |
314/16 |
Mathlib/LinearAlgebra/Span/Defs.lean,Mathlib/RingTheory/DividedPowers/SubDPIdeal.lean |
2 |
1 |
['github-actions'] |
nobody |
10-45519 10 days ago |
10-49753 10 days ago |
10-49804 10 days |
26938 |
JovanGerb author:JovanGerb |
chore(gcongr): set `synthAssignedInstances := false` |
`synthAssignedInstances` is set to false in `congr` and `congr!` (when applying `@[congr]` lemmas). So it is natural to do the same in `gcongr` (when applying `@[gcongr]` lemmas). This should also marginally improve performance.
---
[](https://gitpod.io/from-referrer/)
|
t-meta |
2/1 |
Mathlib/Tactic/GCongr/Core.lean |
1 |
4 |
['JovanGerb', 'github-actions', 'leanprover-bot'] |
nobody |
10-26705 10 days ago |
10-29502 10 days ago |
10-42981 10 days |
26814 |
KiringYJ author:KiringYJ |
feat(MeasureTheory): expose `m.SigmaAlgebra` and `IsSigmaAlgebra` |
(New PR opened because I mis-clicked “Merge” on the previous branch and had to revert it.)
This PR introduces a lightweight API for treating the σ‑algebra of a `MeasurableSpace` as a plain `Set (Set α)`, plus a semantic predicate `IsSigmaAlgebra` and small bridges between bundled and un‑bundled views.
#### Motivation
The immediate goal is to prepare for a formalization of the **monotone class theorem**. With `m.SigmaAlgebra` and the `IsSigmaAlgebra` predicate, one can state the theorem as a clean equality of families of sets, e.g.
```lean
SigmaAlgebra.generateFrom G = MonotoneClass.generateFrom G
```
rather than the more cumbersome phrasing "`s` is measurable ↔ `s` belongs to the smallest monotone class containing `G`". The helpers in this PR make those equalities ergonomic and reusable.
#### What’s new
- **`m.SigmaAlgebra`** – the collection of all `m`‑measurable sets, exposed as a value of type `Set (Set α)`. Lets you write `s ∈ m.SigmaAlgebra` instead of `MeasurableSet[m] s`.
- **`IsSigmaAlgebra F`** – predicate saying that a family of sets `A` is already a σ‑algebra, defined by `(generateFrom F).SigmaAlgebra = F`.
- **`generateFrom_sigmaAlgebra_eq`** – idempotence lemma `generateFrom m.SigmaAlgebra = m` (`@[simp]`).
- Boolean‑algebra instance on `m.SigmaAlgebra` (alias of the existing subtype instance).
- Helper lemmas:
- `Subtype.mem_sigma` – bundled measurable set ∈ `m.SigmaAlgebra`.
- `Set.toMeasurableSubtype` – wrap a membership proof into the subtype.
#### House‑keeping
- Removed two obsolete `noncomputable` keywords from `Mathlib/MeasureTheory/MeasurablyGenerated.lean`; the affected instances are now computable.
#### Notes
- **No breaking changes**: the new definitions are additive; existing code continues to compile unchanged.
- **No dependencies on other PRs**: this patch is self‑contained. |
new-contributor
t-measure-probability
|
86/3 |
Mathlib.lean,Mathlib/MeasureTheory/MeasurableSpace/MeasurablyGenerated.lean,Mathlib/MeasureTheory/MeasurableSpace/SigmaAlgebra.lean |
3 |
1 |
['github-actions'] |
nobody |
9-80538 9 days ago |
13-69507 13 days ago |
13-69552 13 days |
26956 |
mariainesdff author:mariainesdff |
feat(RingTheory/DividedPowers/Basic): add divided power structure on pZp |
We construct a divided power structure on the ideal `(p) ⊆ ℤ_[p]`, given by the family of maps `fun n x ↦ x^n / n!`.
Co-authored-by: @AntoineChambert-Loir
---
[](https://gitpod.io/from-referrer/)
|
|
561/2 |
Mathlib.lean,Mathlib/Data/Nat/Factorial/NatCast.lean,Mathlib/RingTheory/DividedPowers/Padic.lean,Mathlib/RingTheory/DividedPowers/RatAlgebra.lean |
4 |
1 |
['github-actions'] |
nobody |
9-66547 9 days ago |
9-66554 9 days ago |
9-68896 9 days |
26941 |
pechersky author:pechersky |
chore(GroupWithZero/WithZero): use `recZeroCoe` for `WithZero.lift'` |
gives better simps apply lemmas
---
[](https://gitpod.io/from-referrer/)
|
t-order
t-algebra
label:t-algebra$ |
2/4 |
Mathlib/Algebra/GroupWithZero/WithZero.lean |
1 |
3 |
['github-actions', 'kbuzzard', 'pechersky'] |
nobody |
9-44964 9 days ago |
10-38194 10 days ago |
10-38260 10 days |
26881 |
emo916math author:emo916math |
feat(Analysis/Calculus/Deriv/Star) A formula for `deriv (conj ∘ f ∘ conj)` |
Added a lemma that `deriv (conj ∘ f ∘ conj) = conj ∘ deriv f ∘ conj`, proved by cases on whether the derivative mathematically exists or not. This PR replaces [#26805](https://github.com/leanprover-community/mathlib4/pull/26805); see discussion there.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-analysis
|
50/2 |
Mathlib/Analysis/Calculus/Deriv/Star.lean |
1 |
7 |
['emo916math', 'github-actions', 'kckennylau'] |
nobody |
9-32419 9 days ago |
12-29457 12 days ago |
12-29501 12 days |
25931 |
joelriou author:joelriou |
refactor(CategoryTheory): redefine triangulated subcategories using ObjectProperty |
---
This PR continues the work from #24191.
Original PR: https://github.com/leanprover-community/mathlib4/pull/24191 |
|
279/191 |
Mathlib/Algebra/Homology/DerivedCategory/Basic.lean,Mathlib/CategoryTheory/ObjectProperty/ContainsZero.lean,Mathlib/CategoryTheory/ObjectProperty/Shift.lean,Mathlib/CategoryTheory/Triangulated/HomologicalFunctor.lean,Mathlib/CategoryTheory/Triangulated/Subcategory.lean |
5 |
2 |
['github-actions', 'joelriou'] |
nobody |
9-29650 9 days ago |
34-35947 1 month ago |
34-35928 34 days |
26022 |
AntoineChambert-Loir author:AntoineChambert-Loir |
feat(RingTheory/MvPolynomial/Groebner): add docstring and a particular case |
* add a new division theorem when one divides by a single polynomial
* add docstrings to the three division theorems
This PR continues the work from #24819.
Original PR: https://github.com/leanprover-community/mathlib4/pull/24819 |
t-algebra label:t-algebra$ |
27/3 |
Mathlib/RingTheory/MvPolynomial/Groebner.lean |
1 |
2 |
['AntoineChambert-Loir', 'github-actions'] |
nobody |
9-18787 9 days ago |
32-58854 1 month ago |
32-58903 32 days |
26368 |
Whysoserioushah author:Whysoserioushah |
feat(RingTheory/TwoSidedIdeal/SpanAsSum): span of set as finsum |
Reopened after everything moved to fork (#23320).
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
81/0 |
Mathlib.lean,Mathlib/RingTheory/TwoSidedIdeal/SpanAsSum.lean |
2 |
5 |
['github-actions', 'kckennylau'] |
nobody |
9-7591 9 days ago |
25-33710 25 days ago |
25-33756 25 days |
26945 |
gasparattila author:gasparattila |
feat(LinearAlgebra/AffineSpace/AffineSubspace): basic properties of `sInf` and `iInf` |
These properties are analogous to the existing ones for the binary infimum.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-algebra
label:t-algebra$ |
48/1 |
Mathlib/LinearAlgebra/AffineSpace/AffineSubspace/Defs.lean |
1 |
4 |
['Ruben-VandeVelde', 'gasparattila', 'github-actions'] |
nobody |
8-70239 8 days ago |
10-35255 10 days ago |
10-35301 10 days |
26986 |
WangYiran01 author:WangYiran01 |
feat(Partition): add bijection for partitions with max part ≤ r |
## Summary
This PR adds a new theorem `partition_max_equals_bound` to `Mathlib.Combinatorics.Enumerative.Partition`.
It constructs a bijection between:
- The set of partitions of `n` in which `r ∈ π.parts` and all parts are `≤ r`, and
- The set of partitions of `n - r` whose largest part is at most `r`.
This provides a constructive proof via removing/adding `r` from/to the partition multiset, in line with classical enumerative combinatorics.
## Implementation notes
- The proof uses `Multiset.erase` and `Multiset.cons` with basic properties of `sum`, `sup`, and `Partition` structures.
- The bijection is implemented explicitly via `f` and `g`, and proven mutually inverse via `Subtype.ext`.
## Linting
- [x] Passes `lake build`
- [x] Linter clean (no commandStart or longLine issues)
## Author
Contributed by Yiran Wang.
|
new-contributor
t-combinatorics
|
85/0 |
Mathlib/Combinatorics/Enumerative/Partition.lean |
1 |
2 |
['WangYiran01', 'github-actions'] |
nobody |
8-66691 8 days ago |
8-68056 8 days ago |
8-68100 8 days |
26988 |
YaelDillies author:YaelDillies |
feat(Rel): more API |
Some of this API already exists in `Topology.UniformSpace.Defs` but not spelled with `Rel`, some of it was written for #24173.
---
`Topology.UniformSpace.Defs` will be refactored to use these new lemmas in #23181.
[](https://gitpod.io/from-referrer/)
|
t-data |
169/7 |
Mathlib/Combinatorics/SimpleGraph/Basic.lean,Mathlib/Data/Rel.lean |
2 |
1 |
['github-actions'] |
nobody |
8-60028 8 days ago |
8-63853 8 days ago |
8-63904 8 days |
26989 |
joelriou author:joelriou |
feat(CategoryTheory): Artinian objects |
The API for Noetherian objects (from `Subobject.NoetherianObject`) is "dualized" in order to develop an API for Artinian objects. The previously existing definitions `ArtinianObject` and `NoetherianObject` from the file `CategoryTheory.Noetherian` are deprecated.
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-category-theory
|
176/58 |
Mathlib.lean,Mathlib/CategoryTheory/Noetherian.lean,Mathlib/CategoryTheory/Subobject/ArtinianObject.lean,Mathlib/CategoryTheory/Subobject/NoetherianObject.lean |
4 |
1 |
['github-actions', 'javra'] |
nobody |
8-59545 8 days ago |
8-63509 8 days ago |
8-63558 8 days |
26827 |
pechersky author:pechersky |
feat(Analysis/Normed/ValuativeRel): helper instance for NormedField |
---
[](https://gitpod.io/from-referrer/)
- [x] depends on: #26713
- [x] depends on: #26826
|
t-algebra
t-analysis
t-number-theory
label:t-algebra$ |
238/25 |
Mathlib.lean,Mathlib/Analysis/Normed/ValuativeRel.lean,Mathlib/Topology/Algebra/Valued/ValuativeRel.lean |
3 |
11 |
['ADedecker', 'adamtopaz', 'github-actions', 'mathlib4-dependent-issues-bot', 'pechersky'] |
nobody |
8-56991 8 days ago |
12-33817 12 days ago |
12-34081 12 days |
24730 |
YaelDillies author:YaelDillies |
feat(RingTheory): group-like elements |
Define group-like elements in a bialgebra, ie elements such that `η a = 1` and `Δ a = a ⊗ₜ a`.
We prove that group-like elements of a coalgebra over a domain are linearly independent, group-like elements of a bialgebra form a monoid, group-like elements of a Hopf algebra form a group.
From Toric
Co-authored-by: Michał Mrugała
---
- [x] depends on: #24747
[](https://gitpod.io/from-referrer/)
|
toric
t-algebra
label:t-algebra$ |
309/0 |
Mathlib.lean,Mathlib/RingTheory/Bialgebra/GroupLike.lean,Mathlib/RingTheory/Coalgebra/GroupLike.lean,Mathlib/RingTheory/HopfAlgebra/GroupLike.lean |
4 |
33 |
['Julian-Kuelshammer', 'Parcly-Taxel', 'YaelDillies', 'erdOne', 'eric-wieser', 'github-actions', 'leanprover-bot', 'mathlib4-dependent-issues-bot', 'smorel394'] |
nobody |
8-56682 8 days ago |
70-22414 2 months ago |
70-23967 70 days |
26201 |
scholzhannah author:scholzhannah |
feat: subcomplexes of a classical CW complex |
This PR defines subcomplexes of a (classical relative) CW complex to be a closed subspace which is a union of open cells. It provides additional definitions for alternative ways to describe subcomplexes. Lastly, it refactors the definition of the skeleton to define it as a subcomplex.
Co-authored-by: Floris van Doorn
---
[](https://gitpod.io/from-referrer/)
|
t-topology |
213/25 |
Mathlib/Topology/CWComplex/Classical/Basic.lean |
1 |
2 |
['github-actions', 'leanprover-community-bot-assistant'] |
nobody |
8-55969 8 days ago |
8-55991 8 days ago |
27-81331 27 days |
27000 |
gasparattila author:gasparattila |
feat(Analysis/Normed/Group/Quotient): isometric versions of isomorphisms |
This PR adds an isometric version of the third isomorphism theorem for groups and modules.
---
[](https://gitpod.io/from-referrer/)
|
large-import
new-contributor
t-analysis
|
49/2 |
Mathlib/Analysis/Normed/Group/Quotient.lean |
1 |
1 |
['github-actions'] |
nobody |
8-50819 8 days ago |
8-50821 8 days ago |
8-50873 8 days |
23181 |
YaelDillies author:YaelDillies |
refactor(Topology/UniformSpace): use `Rel` |
What's left in `UniformSpace.Defs` is precisely the theory of the uniformity filter.
The motivation is that the theory of coverings and packings in both high dimensional probability and dynamics can be based on entourages, while they have little to do with the uniformity filter (indeed, entourages are in a sense a quantitative version of the uniformity filter).
---
- [x] depends on: #25587
[](https://gitpod.io/from-referrer/)
|
t-topology |
771/587 |
Mathlib/Data/Rel.lean,Mathlib/Dynamics/TopologicalEntropy/CoverEntropy.lean,Mathlib/Dynamics/TopologicalEntropy/DynamicalEntourage.lean,Mathlib/Dynamics/TopologicalEntropy/NetEntropy.lean,Mathlib/Dynamics/TopologicalEntropy/Semiconj.lean,Mathlib/Dynamics/TopologicalEntropy/Subset.lean,Mathlib/InformationTheory/Hamming.lean,Mathlib/MeasureTheory/Measure/RegularityCompacts.lean,Mathlib/Topology/MetricSpace/BundledFun.lean,Mathlib/Topology/MetricSpace/PiNat.lean,Mathlib/Topology/Metrizable/Uniformity.lean,Mathlib/Topology/UniformSpace/Ascoli.lean,Mathlib/Topology/UniformSpace/Basic.lean,Mathlib/Topology/UniformSpace/Cauchy.lean,Mathlib/Topology/UniformSpace/Compact.lean,Mathlib/Topology/UniformSpace/CompactConvergence.lean,Mathlib/Topology/UniformSpace/Completion.lean,Mathlib/Topology/UniformSpace/Defs.lean,Mathlib/Topology/UniformSpace/DiscreteUniformity.lean,Mathlib/Topology/UniformSpace/Equicontinuity.lean,Mathlib/Topology/UniformSpace/HeineCantor.lean,Mathlib/Topology/UniformSpace/OfCompactT2.lean,Mathlib/Topology/UniformSpace/OfFun.lean,Mathlib/Topology/UniformSpace/Separation.lean,Mathlib/Topology/UniformSpace/Ultra/Basic.lean,Mathlib/Topology/UniformSpace/Ultra/Constructions.lean,Mathlib/Topology/UniformSpace/UniformApproximation.lean,Mathlib/Topology/UniformSpace/UniformConvergence.lean,Mathlib/Topology/UniformSpace/UniformEmbedding.lean |
29 |
25 |
['ADedecker', 'PatrickMassot', 'YaelDillies', 'b-mehta', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
8-42336 8 days ago |
8-42336 8 days ago |
51-82326 51 days |
26036 |
joelriou author:joelriou |
feat(CategoryTheory/Functor): pointwise right derived functors |
This PR introduces pointwise right derived functors as particular cases of pointwise left Kan extensions.
---
This PR continues the work from #22490.
Original PR: https://github.com/leanprover-community/mathlib4/pull/22490 |
t-category-theory |
160/0 |
Mathlib.lean,Mathlib/CategoryTheory/Functor/Derived/PointwiseRightDerived.lean |
2 |
2 |
['github-actions', 'joelriou'] |
nobody |
8-41494 8 days ago |
32-49820 1 month ago |
32-49865 32 days |
27008 |
oliver-butterley author:oliver-butterley |
feat(Dynamics): add `comp_iterate_integrable` |
If an observable is integrable then the observable formed by composing with iterates of a measure preserving map is also integrable.
Co-authored-by: Lua Viana Reis me@lua.blog.br
---
[](https://gitpod.io/from-referrer/)
|
t-dynamics |
34/0 |
Mathlib.lean,Mathlib/Dynamics/MeasurePreserving/Lemmas.lean |
2 |
1 |
['github-actions'] |
nobody |
8-39039 8 days ago |
8-39048 8 days ago |
8-39095 8 days |
26660 |
strihanje01 author:strihanje01 |
feat(Combinatorics/Additive/VerySmallDoubling): weak non-commutative Kneser's theorem |
add theorem about the structure of a doubling smaller than the golden ratio
---
[](https://gitpod.io/from-referrer/)
|
large-import
new-contributor
t-combinatorics
|
430/5 |
Mathlib/Combinatorics/Additive/VerySmallDoubling.lean |
1 |
59 |
['YaelDillies', 'github-actions', 'strihanje01'] |
nobody |
8-33617 8 days ago |
8-33617 8 days ago |
13-83837 13 days |
26101 |
xroblot author:xroblot |
feat(NumberField): specialized version of Kummer Dedekind for the splitting of prime numbers |
We prove a specialized version of [KummerDedekind.normalizedFactorsMapEquivNormalizedFactorsMinPolyMk](https://leanprover-community.github.io/mathlib4_docs/Mathlib/NumberTheory/KummerDedekind.html#KummerDedekind.normalizedFactorsMapEquivNormalizedFactorsMinPolyMk) for the splitting of rational prime numbers in number fields.
This PR continues the work from #25038.
---
- [ ] depends on: #26137 |
t-number-theory |
172/2 |
Mathlib/NumberTheory/NumberField/Ideal/KummerDedekind.lean,Mathlib/NumberTheory/RamificationInertia/Basic.lean,Mathlib/RingTheory/AdjoinRoot.lean,Mathlib/RingTheory/DedekindDomain/Ideal.lean,Mathlib/RingTheory/Ideal/Over.lean |
5 |
4 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'xroblot'] |
nobody |
8-20897 8 days ago |
8-20914 8 days ago |
0-50 50 seconds |
25970 |
wwylele author:wwylele |
feat(RingTheory): decompose archimedean classes of HahnSeries |
In preparation for #25140, this connects archimedean class and HahnSeries
---
- [x] depends on: #26773
- [x] depends on: #26787
- [x] depends on: #26788
- [x] depends on: #26789
[](https://gitpod.io/from-referrer/)
|
large-import |
367/2 |
Mathlib/Algebra/Order/Archimedean/Class.lean,Mathlib/RingTheory/HahnSeries/Lex.lean |
2 |
6 |
['ScottCarnahan', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'wwylele'] |
nobody |
8-10425 8 days ago |
8-11958 8 days ago |
26-44551 26 days |
27016 |
Komyyy author:Komyyy |
feat: `⋃ x ∈ s ×ˢ t, f x.1 ×ˢ g x.2 = (⋃ x ∈ s, f x) ×ˢ (⋃ x ∈ t, g x)` etc. |
This lemma is needed to prove that finite product of Alexandrov-discrete spaces is Alexandrov-discrete: #27018
This is the generalization of [Set.iUnion_prod](https://leanprover-community.github.io/mathlib4_docs/Mathlib/Data/Set/Lattice/Image.html#Set.iUnion_prod) to `biUnion`.
Also generalize pi version.
Also generalize the type of the lemma
```lean
`⋃ (i : ι), ⋃ j, ⋃ (i' : ι), ⋃ j', s i j i' j' = ⋃ (i' : ι), ⋃ j', ⋃ (i : ι), ⋃ j, s i j i' j'`
```
to
```lean
`⋃ (i : ι), ⋃ j, ⋃ (i' : ι'), ⋃ j', s i j i' j' = ⋃ (i' : ι'), ⋃ j', ⋃ (i : ι), ⋃ j, s i j i' j'`
```
---
Caution: The generalization of this lemma to `⋂` is not easy because it requires nonempty.
[](https://gitpod.io/from-referrer/)
|
t-set-theory |
19/4 |
Mathlib/Data/Set/Lattice.lean,Mathlib/Data/Set/Lattice/Image.lean |
2 |
1 |
['github-actions'] |
nobody |
7-85382 7 days ago |
8-2299 8 days ago |
8-3474 8 days |
27019 |
Komyyy author:Komyyy |
feat: T1 Alexandrov-discrete topology is discrete |
---
[](https://gitpod.io/from-referrer/)
|
t-topology |
24/0 |
Mathlib.lean,Mathlib/Topology/Separation/AlexandrovDiscrete.lean |
2 |
1 |
['github-actions'] |
nobody |
7-82875 7 days ago |
7-83177 7 days ago |
7-83161 7 days |
25899 |
pfaffelh author:pfaffelh |
feat(Topology/Compactness/CompactSystem): introduce compact Systems |
A compact system is a set systems with the property that, whenever a countable intersections of sets in the set system is empty, there is a finite subset of sets with empty intersection. These are needed e.g. in measure theory if one wants to show sigma-additivity of a set function on a ring.
* Main result: The set of sets which are either compact and closed, or `univ`, is a compact system.
* Introduce `Dissipate s x := ⋂ y ≤ x, s y` (Data/Set/Dissipate), which is parallel to Data/Set/Accumulate.
Co-authored-by: Rémy Degenne remydegenne@gmail.com
---
*This PR continues the work from #24541.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/24541* |
t-topology |
453/2 |
Mathlib.lean,Mathlib/Data/Set/Accumulate.lean,Mathlib/Data/Set/Dissipate.lean,Mathlib/MeasureTheory/PiSystem.lean,Mathlib/Topology/Compactness/CompactSystem.lean |
5 |
1 |
['github-actions'] |
nobody |
7-76692 7 days ago |
7-76692 7 days ago |
34-59388 34 days |
26272 |
ajirving author:ajirving |
feat(NumberTheory/LucasLehmer): prove converse direction to Lucas-Lehmer |
Proves the converse direction of the Lucas-Lehmer test, namely that the Lucas-Lehmer criterion is a necessary condition for a Mersenne prime.
Adds a couple of examples of proving Mersenne numbers are composite using this.
Proves that if `2^p-1` is prime then `p` is prime.
---
* I wasn't sure how many examples to add given that there are many more Mersenne composites than primes.
* There are a number of annoying coercions between different rings, any simplifications will be appreciated.
[](https://gitpod.io/from-referrer/)
|
large-import
new-contributor
t-number-theory
|
226/5 |
Archive/Examples/MersennePrimes.lean,Mathlib/NumberTheory/LucasLehmer.lean |
2 |
12 |
['github-actions', 'kckennylau'] |
nobody |
7-76654 7 days ago |
27-46075 27 days ago |
27-46121 27 days |
26838 |
vlad902 author:vlad902 |
feat: add lemmas about `List.scanr` |
This PR continues the work from #25188.
Original PR: https://github.com/leanprover-community/mathlib4/pull/25188 |
t-data |
84/19 |
Mathlib/Data/List/Scan.lean |
1 |
12 |
['github-actions', 'vihdzp', 'vlad902'] |
nobody |
7-72719 7 days ago |
12-75228 12 days ago |
12-75282 12 days |
24015 |
alreadydone author:alreadydone |
feat(RingTheory): lemmas on finiteness of `LinearMap` and `Module.End` |
---
One less lemma than #24012, but with the advantage of not depending on #23963.
- [x] depends on: #24115
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
137/81 |
Mathlib/Algebra/Module/LinearMap/End.lean,Mathlib/GroupTheory/GroupAction/SubMulAction.lean,Mathlib/LinearAlgebra/BilinearMap.lean,Mathlib/LinearAlgebra/Dual/Lemmas.lean,Mathlib/LinearAlgebra/Projection.lean,Mathlib/RingTheory/Finiteness/Basic.lean,Mathlib/RingTheory/SimpleModule/Basic.lean |
7 |
19 |
['alreadydone', 'erdOne', 'eric-wieser', 'github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'leanprover-community-mathlib4-bot', 'mathlib4-dependent-issues-bot'] |
erdOne assignee:erdOne |
7-72038 7 days ago |
53-15545 1 month ago |
95-49287 95 days |
25949 |
themathqueen author:themathqueen |
feat(LinearAlgebra/Basis/MulOpposite): basis of an opposite space |
This adds the definition of `Basis.mulOpposite` and shows finite-dimensionality and freeness of `Hᵐᵒᵖ`.
For motivation, see #25951.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-algebra
label:t-algebra$ |
48/0 |
Mathlib.lean,Mathlib/LinearAlgebra/Basis/MulOpposite.lean |
2 |
4 |
['github-actions', 'j-loreaux', 'themathqueen'] |
nobody |
7-50407 7 days ago |
7-50422 7 days ago |
24-75545 24 days |
27030 |
YaelDillies author:YaelDillies |
refactor: use `Algebra.FiniteType` as a class |
Assumptions are currently being passed explicitly, which is quite odd.
Also generalise the ~lemmas~ instances about `Polynomial`, `MvPolynomial`, etc... to be about two rings instead of one.
From Toric
---
[](https://gitpod.io/from-referrer/)
|
toric
t-algebra
label:t-algebra$ |
53/46 |
Mathlib/RingTheory/AdjoinRoot.lean,Mathlib/RingTheory/Extension/Cotangent/Basic.lean,Mathlib/RingTheory/FiniteType.lean |
3 |
1 |
['github-actions'] |
nobody |
7-49215 7 days ago |
7-50838 7 days ago |
7-50833 7 days |
27042 |
Ruben-VandeVelde author:Ruben-VandeVelde |
feat: some WithZero lemmas |
Co-authored-by: matthewjasper <20113453+matthewjasper@users.noreply.github.com>
Co-authored-by: Salvatore Mercuri
---
[](https://gitpod.io/from-referrer/)
|
FLT
t-algebra
label:t-algebra$ |
54/1 |
Mathlib/Algebra/Order/GroupWithZero/Canonical.lean |
1 |
1 |
['github-actions'] |
nobody |
7-31396 7 days ago |
7-31405 7 days ago |
7-31450 7 days |
25786 |
Parcly-Taxel author:Parcly-Taxel |
feat: IMO 2001 Q4 |
|
IMO |
138/4 |
Archive.lean,Archive/Imo/Imo2001Q4.lean,Mathlib/Logic/Equiv/Fin/Rotate.lean |
3 |
6 |
['Parcly-Taxel', 'dwrensha', 'github-actions', 'leanprover-community-bot-assistant'] |
nobody |
6-83352 6 days ago |
13-11219 13 days ago |
35-76791 35 days |
27047 |
YaelDillies author:YaelDillies |
feat: `MonoidHom.toAdditive''` as a `MulEquiv` |
From Toric
---
I haven't yet been very thorough with the new lemmas. I first want to hear thoughts about the names
[](https://gitpod.io/from-referrer/)
|
toric
t-algebra
label:t-algebra$ |
31/7 |
Mathlib/Algebra/Group/TypeTags/Hom.lean |
1 |
1 |
['github-actions'] |
nobody |
6-78294 6 days ago |
6-78311 6 days ago |
7-23768 7 days |
27060 |
YaelDillies author:YaelDillies |
feat: missing definitional lemmas for the braiding on `Mon_ C` |
From Toric
---
[](https://gitpod.io/from-referrer/)
|
toric
t-category-theory
easy
|
3/0 |
Mathlib/CategoryTheory/Monoidal/Mon_.lean |
1 |
1 |
['github-actions'] |
nobody |
6-77584 6 days ago |
6-77637 6 days ago |
6-77638 6 days |
26839 |
kebekus author:kebekus |
feat: implement the Cauchy-Riemann Equation |
Describe complex differentiability for functions `f : ℂ → ℂ` using the Cauchy-Riemann equation.
This material closes a long-standing open TODO. It is used in [Project VD](https://github.com/kebekus/ProjectVD), which aims to formalize Value Distribution Theory for meromorphic functions on the complex plane. It is one of the ingredients in the proof of Jensen's Formula in complex analysis.
---
[](https://gitpod.io/from-referrer/)
|
t-analysis |
125/1 |
Mathlib/Analysis/Complex/Conformal.lean |
1 |
20 |
['YaelDillies', 'github-actions', 'kebekus', 'sgouezel'] |
nobody |
6-75727 6 days ago |
6-75727 6 days ago |
9-83843 9 days |
27064 |
YaelDillies author:YaelDillies |
feat: considering an iso over `S` as an iso in `Over S` |
From Toric
---
[](https://gitpod.io/from-referrer/)
|
toric
t-category-theory
|
41/1 |
Mathlib/CategoryTheory/Comma/Over/OverClass.lean |
1 |
1 |
['github-actions'] |
nobody |
6-74586 6 days ago |
6-74640 6 days ago |
6-74637 6 days |
27031 |
YaelDillies author:YaelDillies |
feat: `Spec(R)` notation for `Spec (CommRingCat.of R)` |
This notation was instrumental in understanding the "industrial size" goals that showed up in Toric. Indeed, `Spec (.of R)` is reasonably short, but it currently pretty-prints as `Spec (CommRingCat.of R)`, which is unbearably long.
There is a slight potential for ambiguity with `Spec R`, which I have hopefully mitigated with a docstring. If ever someone nonetheless writes a lemma about `Spec(R)` where `R : CommRingCat`, all odds are that it will be innocuous since `.of ↑R = R` definitionally.
Alternatively, we could make the `Spec(R)` notation and delaborator automatically detect whether `R : CommRingCat` or not. I would rather postpone this extra complexity until strictly necessary.
From Toric
---
[](https://gitpod.io/from-referrer/)
|
toric
t-algebraic-geometry
|
73/62 |
Mathlib/AlgebraicGeometry/AffineScheme.lean,Mathlib/AlgebraicGeometry/AffineSpace.lean,Mathlib/AlgebraicGeometry/Cover/Open.lean,Mathlib/AlgebraicGeometry/IdealSheaf/Subscheme.lean,Mathlib/AlgebraicGeometry/Limits.lean,Mathlib/AlgebraicGeometry/Modules/Tilde.lean,Mathlib/AlgebraicGeometry/Morphisms/ClosedImmersion.lean,Mathlib/AlgebraicGeometry/Morphisms/FiniteType.lean,Mathlib/AlgebraicGeometry/Morphisms/Proper.lean,Mathlib/AlgebraicGeometry/Morphisms/UniversallyClosed.lean,Mathlib/AlgebraicGeometry/Noetherian.lean,Mathlib/AlgebraicGeometry/OpenImmersion.lean,Mathlib/AlgebraicGeometry/PointsPi.lean,Mathlib/AlgebraicGeometry/ProjectiveSpectrum/Basic.lean,Mathlib/AlgebraicGeometry/ProjectiveSpectrum/Proper.lean,Mathlib/AlgebraicGeometry/Pullbacks.lean,Mathlib/AlgebraicGeometry/ResidueField.lean,Mathlib/AlgebraicGeometry/Restrict.lean,Mathlib/AlgebraicGeometry/Scheme.lean,Mathlib/AlgebraicGeometry/Stalk.lean,Mathlib/AlgebraicGeometry/ValuativeCriterion.lean |
21 |
5 |
['YaelDillies', 'edegeltje', 'github-actions'] |
nobody |
6-73540 6 days ago |
7-49504 7 days ago |
7-49504 7 days |
24527 |
matthewjasper author:matthewjasper |
feat(Topology/Algebra/Module): Add more theorems for IsModuleTopology |
Add theorems that surjective linear maps to the module topology are open.
Add IsModuleTopology instance for quotients.
Add IsModuleTopology instance for finite dimensional T2 vector spaces over a complete normed field and use it to shorten some proofs.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-algebra
t-topology
label:t-algebra$ |
48/24 |
Mathlib/Topology/Algebra/Module/FiniteDimension.lean,Mathlib/Topology/Algebra/Module/ModuleTopology.lean |
2 |
7 |
['erdOne', 'github-actions', 'matthewjasper', 'riccardobrasca'] |
nobody |
6-57126 6 days ago |
77-59741 2 months ago |
79-28037 79 days |
26580 |
vasnesterov author:vasnesterov |
feat(Tactic/Order): translate linear orders to `Int` |
It was [pointed out](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/tactic.20for.20partial.20orders/near/515897754) that `order` is not complete for linear orders with lattice operations (while it remains complete for linear orders without lattice operations and for general lattices without assuming linearity). The problem for linear orders with lattice operations is NP-hard, but it can be translated from an arbitrary type to `Int` and then solved using a smart and efficient procedure (such as `omega`). This PR implements such a translation within the `order` tactic.
Co-authored-by: Aaron Liu
---
- [x] depends on: #26354
[](https://gitpod.io/from-referrer/) |
large-import
t-meta
|
302/22 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Order.lean,Mathlib/Tactic/Order/Graph/Basic.lean,Mathlib/Tactic/Order/Preprocessing.lean,Mathlib/Tactic/Order/ToInt.lean,MathlibTest/order.lean |
7 |
4 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'vasnesterov'] |
nobody |
6-54459 6 days ago |
6-66367 6 days ago |
6-68067 6 days |
26899 |
robin-carlier author:robin-carlier |
feat(CategoryTheory/Functor/KanExtension): transitivity of left Kan extensions |
In this PR, we show that left Kan extensions are "transitive" in the following sense : if `α : F₀ ⟶ L ⋙ F₁` exhibits `F₁` as a left Kan extension of `F₀` along `L : C ⥤ D`, then given a functor `L' : D ⥤ D'` an an extension `(β : F₁ ⟶ L' ⋙ F₂)`, the "pasted extension" formed by `α` and `β` exhibits `F₂` as a left Kan extension of `F₀` along `L ⋙ L'` if and only if `β` exhibits `F₂` as a left Kan extension of `F₁` along `L'`. This refines the current theorems in mathlib that only treat the case where we pre or post-compose by an equivalence.
The actual statement we prove is "fully weak" and lets us pick a functor isomorphic to `L ⋙ L'` and an extension isomorphic to the pasted one if needed.
---
I will PR the dual version of everything for right Kan extensions as soon as we settle on the final form of this one.
[](https://gitpod.io/from-referrer/)
|
t-category-theory |
144/0 |
Mathlib/CategoryTheory/Functor/KanExtension/Basic.lean |
1 |
8 |
['github-actions', 'joelriou', 'robin-carlier'] |
nobody |
6-52370 6 days ago |
6-52370 6 days ago |
9-23600 9 days |
26640 |
euprunin author:euprunin |
chore: golf Data/ using `grind` |
|
bench-after-CI
t-data
|
14/91 |
Mathlib/Data/EReal/Operations.lean,Mathlib/Data/List/Cycle.lean,Mathlib/Data/List/Indexes.lean,Mathlib/Data/List/Induction.lean,Mathlib/Data/List/Nodup.lean,Mathlib/Data/List/Permutation.lean,Mathlib/Data/List/Sigma.lean,Mathlib/Data/PEquiv.lean,Mathlib/Data/PNat/Xgcd.lean,Mathlib/Data/Prod/Lex.lean,Mathlib/Data/Seq/Parallel.lean,Mathlib/Data/Set/Lattice.lean |
12 |
12 |
['euprunin', 'github-actions', 'grunweg', 'leanprover-bot', 'leanprover-community-mathlib4-bot'] |
nobody |
6-27256 6 days ago |
6-27306 6 days ago |
17-28731 17 days |
27095 |
themathqueen author:themathqueen |
feat(Algebra/Star/SelfAdjoint): some API for `IsStarNormal` |
This adds api for adding and subtracting normal elements.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
24/3 |
Mathlib/Algebra/Star/SelfAdjoint.lean |
1 |
2 |
['eric-wieser', 'github-actions'] |
nobody |
6-21831 6 days ago |
6-27648 6 days ago |
6-27694 6 days |
27049 |
BoltonBailey author:BoltonBailey |
doc(Analysis/BoxIntegral/Partition/Filter): field docstrings |
Split of #25917. Adds docstrings to the fields of this structure (Taken from the docstring of the structure itself). Note: this documentation was originally changed by asking Cursor (Claude 3.5 sonnet) to write the docstrings, but I think ultimately the docstring of the struct was reworked.
---
[](https://gitpod.io/from-referrer/)
|
t-analysis |
13/14 |
Mathlib/Analysis/BoxIntegral/Partition/Filter.lean |
1 |
2 |
['BoltonBailey', 'github-actions'] |
nobody |
6-17873 6 days ago |
7-20365 7 days ago |
7-20585 7 days |
26968 |
vihdzp author:vihdzp |
feat(Order/Concept): sets in a concept are codisjoint |
...and other small lemmata.
---
- [x] depends on: #26976
[](https://gitpod.io/from-referrer/)
|
t-order |
33/2 |
Mathlib/Order/Concept.lean |
1 |
8 |
['github-actions', 'leanprover-community-bot-assistant', 'linesthatinterlace', 'mathlib4-dependent-issues-bot', 'plp127', 'vihdzp'] |
nobody |
6-15581 6 days ago |
6-15597 6 days ago |
6-45149 6 days |
27073 |
pechersky author:pechersky |
feat(Archive/Examples/Local): files showcasing properties of local fields |
for p-adics, completions of number fields, laurent series, and fraction rings of witt vectors
Should get filled in as more data/instances are declared
---
[](https://gitpod.io/from-referrer/)
|
|
139/0 |
Archive.lean,Archive/Examples/Local/Laurent.lean,Archive/Examples/Local/NumberField.lean,Archive/Examples/Local/Padic.lean,Archive/Examples/Local/Witt.lean |
5 |
1 |
['github-actions'] |
nobody |
6-8740 6 days ago |
6-49310 6 days ago |
6-49292 6 days |
27110 |
pechersky author:pechersky |
chore(Valued/WithVal): apply_symm_equiv |
valuation on the WIthVal is equal to the underlying valuation and simp tag
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-topology
t-number-theory
easy
label:t-algebra$ |
4/0 |
Mathlib/Topology/Algebra/Valued/WithVal.lean |
1 |
1 |
['github-actions'] |
nobody |
6-325 6 days ago |
6-328 6 days ago |
6-382 6 days |
27109 |
pechersky author:pechersky |
feat(RingTheory/AdicValuation): valuation_surjective |
for both the base valuation and the one on the extension
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-analysis
t-number-theory
label:t-algebra$ |
31/0 |
Mathlib/RingTheory/DedekindDomain/AdicValuation.lean,Mathlib/Topology/Algebra/Valued/ValuedField.lean |
2 |
1 |
['github-actions'] |
nobody |
6-315 6 days ago |
6-315 6 days ago |
6-396 6 days |
27116 |
pechersky author:pechersky |
feat(Valued): FaithfulSMul to completion |
simplifies coercions and golfs existing instance
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-analysis
t-number-theory
label:t-algebra$ |
24/6 |
Mathlib/RingTheory/DedekindDomain/AdicValuation.lean,Mathlib/Topology/Algebra/Valued/ValuedField.lean |
2 |
1 |
['github-actions'] |
nobody |
5-81455 5 days ago |
5-81509 5 days ago |
5-81510 5 days |
25814 |
vlad902 author:vlad902 |
feat(SimpleGraph): Weaker condition for paths in acyclic graphs |
`IsAcyclic.isPath_iff_chain'` defines a weaker condition for proving that a walk is a path, in particular it shows that rather than proving that all vertices in the support of a walk are distinct, one must only show that consecutive edges are distinct (e.g. every other vertex must be distinct.) This leads to a simple corollary that trails are also paths in acyclic graphs.
I had a need for this when formalizing Cayley graphs, since this condition maps cleanly onto words in free groups being reduced.
---
*This PR continues the work from #25630.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/25630* |
t-combinatorics |
43/0 |
Mathlib/Combinatorics/SimpleGraph/Acyclic.lean,Mathlib/Combinatorics/SimpleGraph/Paths.lean |
2 |
2 |
['github-actions', 'vlad902'] |
nobody |
5-80353 5 days ago |
37-50281 1 month ago |
37-50264 37 days |
27120 |
YaelDillies author:YaelDillies |
feat: the category of commutative bialgebras |
Define the bundled category `CommBialgCat R` of commutative bialgebras over a fixed commutative ring `R` along with the forgetful functor to `CommAlgCat`.
From Toric
Co-authored-by: Andrew Yang
Co-authored-by: Michał Mrugała
---
[](https://gitpod.io/from-referrer/)
|
toric
t-algebra
label:t-algebra$ |
235/0 |
Mathlib.lean,Mathlib/Algebra/Category/CommBialgCat.lean |
2 |
1 |
['github-actions'] |
nobody |
5-77189 5 days ago |
5-77189 5 days ago |
5-77259 5 days |
26782 |
euprunin author:euprunin |
chore: golf Algebra/ using `exact` |
|
t-algebra label:t-algebra$ |
67/172 |
Mathlib/Algebra/Algebra/Spectrum/Basic.lean,Mathlib/Algebra/BigOperators/Finprod.lean,Mathlib/Algebra/BigOperators/Group/Finset/Basic.lean,Mathlib/Algebra/ContinuedFractions/Computation/Translations.lean,Mathlib/Algebra/CubicDiscriminant.lean,Mathlib/Algebra/GCDMonoid/Basic.lean,Mathlib/Algebra/Group/Fin/Basic.lean,Mathlib/Algebra/GroupWithZero/NonZeroDivisors.lean,Mathlib/Algebra/Homology/Embedding/Extend.lean,Mathlib/Algebra/Homology/HomologicalComplexAbelian.lean,Mathlib/Algebra/Homology/HomotopyCategory/ShiftSequence.lean,Mathlib/Algebra/Homology/ShortComplex/ConcreteCategory.lean,Mathlib/Algebra/Homology/ShortComplex/Exact.lean,Mathlib/Algebra/Homology/ShortComplex/PreservesHomology.lean,Mathlib/Algebra/Homology/ShortComplex/QuasiIso.lean,Mathlib/Algebra/IsPrimePow.lean,Mathlib/Algebra/Lie/CartanExists.lean,Mathlib/Algebra/Lie/Subalgebra.lean,Mathlib/Algebra/Module/FinitePresentation.lean,Mathlib/Algebra/MonoidAlgebra/Defs.lean,Mathlib/Algebra/MonoidAlgebra/NoZeroDivisors.lean,Mathlib/Algebra/MvPolynomial/Rename.lean,Mathlib/Algebra/Order/Group/Abs.lean,Mathlib/Algebra/Order/Ring/Unbundled/Rat.lean,Mathlib/Algebra/Order/Ring/WithTop.lean,Mathlib/Algebra/Polynomial/Coeff.lean,Mathlib/Algebra/Polynomial/Degree/Lemmas.lean,Mathlib/Algebra/Polynomial/Expand.lean,Mathlib/Algebra/Polynomial/Monic.lean,Mathlib/Algebra/Polynomial/Smeval.lean,Mathlib/Algebra/PresentedMonoid/Basic.lean,Mathlib/Algebra/RingQuot.lean,Mathlib/Algebra/Star/Pointwise.lean |
33 |
9 |
['euprunin', 'github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'leanprover-community-mathlib4-bot'] |
nobody |
5-75177 5 days ago |
7-76310 7 days ago |
14-60563 14 days |
24192 |
alreadydone author:alreadydone |
feat(RingTheory): semisimple Wedderburn–Artin existence |
---
- [x] depends on: #24119
- [x] depends on: #23963
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
468/66 |
Mathlib/Algebra/Algebra/Pi.lean,Mathlib/Algebra/Ring/Equiv.lean,Mathlib/LinearAlgebra/DFinsupp.lean,Mathlib/Order/CompleteSublattice.lean,Mathlib/RingTheory/SimpleModule/Basic.lean,Mathlib/RingTheory/SimpleModule/IsAlgClosed.lean,Mathlib/RingTheory/SimpleModule/Isotypic.lean,Mathlib/RingTheory/SimpleModule/WedderburnArtin.lean,docs/1000.yaml |
9 |
4 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
5-71367 5 days ago |
14-64073 14 days ago |
63-14760 63 days |
26464 |
joelriou author:joelriou |
feat(LinearAlgebra): generators of pi tensor products |
In this PR, we show that the `R`-module `⨂[R] i, M i` is finitely generated if the index type is finite and all `M i` are finitely generated. This follows from a more precise result about generators of `⨂[R] i, M i`.
---
This PR continues the work from #18725.
Original PR: https://github.com/leanprover-community/mathlib4/pull/18725 |
file-removed
t-algebra
label:t-algebra$ |
268/4 |
Mathlib.lean,Mathlib/Analysis/NormedSpace/PiTensorProduct/ProjectiveSeminorm.lean,Mathlib/Data/SubtypeNeLift.lean,Mathlib/LinearAlgebra/PiTensorProduct/Basic.lean,Mathlib/LinearAlgebra/PiTensorProduct/Finite.lean,Mathlib/LinearAlgebra/PiTensorProduct/Generators.lean,Mathlib/LinearAlgebra/TensorPower/Basic.lean,Mathlib/RingTheory/PiTensorProduct.lean,Mathlib/SetTheory/Cardinal/Finite.lean |
9 |
10 |
['eric-wieser', 'github-actions', 'joelriou', 'leanprover-community-bot-assistant'] |
nobody |
5-67855 5 days ago |
12-71115 12 days ago |
19-23513 19 days |
27126 |
YaelDillies author:YaelDillies |
chore(CategoryTheory/Monoidal): unify `mkIso` |
Previously, `mkIso` and `mkIso'` meant different things across the various types of objects. Now:
* `mkIso'` takes in elements `X`, `Y` of the underlying category `C`, an isomorphism `e : X ≅ Y` and a typeclass assumption `[IsMon_Hom e.hom]` and returns `mk X ≅ mk Y`,
* `mkIso` is an `abbrev` for `mkIso'`, taking in elements `X`, `Y` of `Obj C`, an isomorphism `e : X.X ≅ Y.X` and the proof fields of `IsMon_Hom e.hom` and returns `X ≅ Y`.
From Toric
---
[](https://gitpod.io/from-referrer/)
|
toric
t-category-theory
|
66/66 |
Mathlib/CategoryTheory/Monoidal/Bimon_.lean,Mathlib/CategoryTheory/Monoidal/CommGrp_.lean,Mathlib/CategoryTheory/Monoidal/CommMon_.lean,Mathlib/CategoryTheory/Monoidal/Grp_.lean,Mathlib/CategoryTheory/Monoidal/Mon_.lean |
5 |
1 |
['github-actions'] |
nobody |
5-62047 5 days ago |
5-62592 5 days ago |
5-62585 5 days |
26623 |
mariainesdff author:mariainesdff |
feat(RingTheory/Valuation/Discrete/Basic): relate DVRs and discrete valuations |
We prove that the valuation subring of a discretely-valued field is a DVR.
Conversely, given a DVR `A` and a field `K` satisfying `IsFractionRing A K`, we show that the valuation induced on `K` is discrete.
We provide the ring isomorphism between a DVR and the valuation subring in its field of fractions endowed with the adic valuation of the maximal ideal.
Co-authored-by: @faenuccio
---
- [ ] depends on: #26591
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebra
label:t-algebra$ |
118/3 |
Mathlib/GroupTheory/SpecificGroups/Cyclic.lean,Mathlib/RingTheory/Valuation/Discrete/Basic.lean |
2 |
5 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
5-61300 5 days ago |
5-61307 5 days ago |
8-44738 8 days |
26955 |
mariainesdff author:mariainesdff |
feat(LinearAlgebra/OnSup): extend linear maps to sums of modules |
Let `A` be a ring, `X, Y` be `A`-modules, and `M, N` be `A`-submodules of `X`.
Given two linear maps `f : M →ₗ[A] Y` and `g : N →ₗ[A] Y` that agree on `M ∩ N`, there is a unique linear map `M + N →ₗ[A] Y` that simultaneously extends `f` and `g`.
Co-authored-by: @AntoineChambert-Loir
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
153/0 |
Mathlib.lean,Mathlib/LinearAlgebra/OnSup.lean |
2 |
15 |
['AntoineChambert-Loir', 'eric-wieser', 'github-actions', 'wwylele'] |
nobody |
5-60736 5 days ago |
5-60803 5 days ago |
6-25310 6 days |
26961 |
mariainesdff author:mariainesdff |
feat(RingTheory/PowerSeries/Substitution): add API |
Co-authored-by: @AntoineChambert-Loir
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
62/1 |
Mathlib/RingTheory/PowerSeries/Basic.lean,Mathlib/RingTheory/PowerSeries/Substitution.lean |
2 |
5 |
['Ruben-VandeVelde', 'github-actions', 'mariainesdff'] |
nobody |
5-57614 5 days ago |
9-63236 9 days ago |
9-63286 9 days |
26106 |
mbkybky author:mbkybky |
feat(RingTheory/Regular): flat base change of weakly regular sequence |
Show that [RingTheory.Sequence.IsWeaklyRegular](https://leanprover-community.github.io/mathlib4_docs/Mathlib/RingTheory/Regular/RegularSequence.html#RingTheory.Sequence.IsWeaklyRegular) is stable under flat base change and [RingTheory.Sequence.IsRegular](https://leanprover-community.github.io/mathlib4_docs/Mathlib/RingTheory/Regular/RegularSequence.html#RingTheory.Sequence.IsRegular) is stable under faithfully flat base change.
Co-authored-by: Nailin Guan @Thmoas-Guan
- [x] depends on: #26297
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
200/6 |
Mathlib.lean,Mathlib/RingTheory/Flat/Basic.lean,Mathlib/RingTheory/Flat/FaithfullyFlat/Basic.lean,Mathlib/RingTheory/IsTensorProduct.lean,Mathlib/RingTheory/Regular/Flat.lean |
5 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
5-54442 5 days ago |
17-66392 17 days ago |
17-66478 17 days |
27059 |
Komyyy author:Komyyy |
feat: Linear upper or lower sets topologies are completely normal |
The primary motivation for this theorem is to prove that Sierpiński space is completely normal.
---
[](https://gitpod.io/from-referrer/)
|
t-topology |
77/1 |
Mathlib.lean,Mathlib/Topology/Order/UpperLowerSetTopology.lean,Mathlib/Topology/Separation/LinearUpperLowerSetTopology.lean |
3 |
1 |
['github-actions'] |
nobody |
5-53605 5 days ago |
6-78030 6 days ago |
6-78013 6 days |
26879 |
robin-carlier author:robin-carlier |
feat(CategoryTheory/Monoidal/DayConvolution): Internal homs for Day convolution |
In this PR, we introduce a structure `DayConvolutionInternalHom` on triples of functors `F G H: C ⥤ V` and that bundles data necessary to exhibit `H` as the value at `G` of an "internal hom functor for F" for the day convolution monoidal structure.
More precisely, under the assumption that `V` is monoidal closed, the required data is that of suitably functorial (in `c` and `G`) ends of the profunctors `c₁ c₂ ↦ ihom (F c₁) (G.obj (c₂ ⊗ c))`. With this data, we construct for every `G` (and for implicit data of relevant day convolutions) transformations `F ⊛ [F, G] ⟶ G` and `G ⟶ [F, (F ⊛ G)]` that one should think of as the components of "evaluations" and "coevaluations" transformations exhibiting `[F, -]` as a right adjoint to `F ⊛ -`. To give body to this claim, we prove that these transformations are natural in `G`, and prove that they satisfy the triangle identities.
This will be used in conjuction with #26820 to show that Day convolution structure are closed whenever `V` is closed and has relevant limits.
---
[](https://gitpod.io/from-referrer/)
|
t-category-theory |
283/1 |
Mathlib.lean,Mathlib/CategoryTheory/Monoidal/DayConvolution.lean,Mathlib/CategoryTheory/Monoidal/DayConvolution/Closed.lean |
3 |
1 |
['github-actions'] |
nobody |
5-53140 5 days ago |
6-54751 6 days ago |
12-21519 12 days |
27076 |
Komyyy author:Komyyy |
refactor: don't require `DecidablePred` to state `PrimrecPred` |
```lean
def PrimrecPred {α} [Primcodable α] (p : α → Prop) [DecidablePred p] :=
Primrec fun a => decide (p a)
```
Currently, `DecidablePred` is required to **state** `PrimrecPred`, so this PR changes the definition and adds convenient APIs for this new definition:
```lean
def PrimrecPred {α} [Primcodable α] (p : α → Prop) :=
open scoped Classical in Primrec fun a => decide (p a)
```
---
[](https://gitpod.io/from-referrer/)
|
t-computability |
117/67 |
Mathlib/Computability/Halting.lean,Mathlib/Computability/Partrec.lean,Mathlib/Computability/Primrec.lean,Mathlib/Computability/Reduce.lean |
4 |
4 |
['Komyyy', 'eric-wieser', 'github-actions'] |
nobody |
5-52512 5 days ago |
6-45704 6 days ago |
6-45689 6 days |
27082 |
staroperator author:staroperator |
feat(Order/WellFoundedSet): add `Set.IsPWO.exists_le_minimal`, `Set.IsPWO.exists_minimal`, `Set.IsPWO.exists_minimalFor` |
which are the `IsPWO` version of `exists_minimal_le_of_wellFoundedLT` and others.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-order
|
22/0 |
Mathlib/Order/WellFoundedSet.lean |
1 |
4 |
['alreadydone', 'github-actions', 'staroperator'] |
nobody |
5-49705 5 days ago |
6-40356 6 days ago |
6-40401 6 days |
27067 |
robin-carlier author:robin-carlier |
feat(CategoryTheory/Monoidal/DayConvolution): braiding and symmetry for Day convolution |
In this PR, we prove that when `C` and `V` are braided monoidal categories, and when relevant Day convolutions exist, the unbundled Day convolution monoidal structure on `C ⥤ V` is also braided: we construct an isomorphism `DayConvolution.braiding`, characterize it with respect to the unit maps that exhibits Day convolutions as left Kan extensions, and prove that the forward and reverse hexagon identities are satisfied.
In the case `C` and `V` are symmetric, we show that `braiding F G|>.hom` is inverse to `braiding G F|>.hom` as well.
---
[](https://gitpod.io/from-referrer/)
|
t-category-theory |
201/1 |
Mathlib.lean,Mathlib/CategoryTheory/Monoidal/DayConvolution.lean,Mathlib/CategoryTheory/Monoidal/DayConvolution/Braided.lean |
3 |
1 |
['github-actions'] |
nobody |
5-48732 5 days ago |
6-67048 6 days ago |
6-67091 6 days |
27003 |
eric-wieser author:eric-wieser |
chore: use `Simp.ResultQ` more often |
Also uses `~q` in place of manual `isDefEq` matching.
---
[](https://gitpod.io/from-referrer/)
|
t-meta |
18/22 |
Mathlib/Tactic/NormNum/Core.lean,Mathlib/Tactic/NormNum/Result.lean,Mathlib/Tactic/ReduceModChar.lean |
3 |
2 |
['eric-wieser', 'github-actions'] |
nobody |
5-47913 5 days ago |
8-46140 8 days ago |
8-46123 8 days |
26851 |
oliver-butterley author:oliver-butterley |
feat(Mathlib/Algebra/Order): add 3 lemmas related to `partialSups` |
Add 3 lemmas related to `partialSups`:
- One concerns the partialSup of a function with a constant added
- Two concern the partialSup of the succ, both of which are natural variants of the other lemma already mathlib.
The lemmas couldn't be added to any of the files which already contain similar results on `partialSups` because in each case it would significantly increase imports.
Are these lemmas correctly located? Another option would be to have a folder `PartialSups` containing multiple files with the different lemmas.
- [x] depends on: #26848
Co-authored-by: Lua Viana Reis
---
[](https://gitpod.io/from-referrer/)
|
t-order |
58/0 |
Mathlib.lean,Mathlib/Algebra/Order/AddGroup/PartialSups.lean,Mathlib/Algebra/Order/SuccOrder/PartialSups.lean |
3 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
5-47639 5 days ago |
5-47639 5 days ago |
5-54764 5 days |
27108 |
pechersky author:pechersky |
chore(RingTheory/AdicValuation): golf using WithZero.log |
with helper lemma of how `log` preserves order
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-number-theory
label:t-algebra$ |
15/16 |
Mathlib/Algebra/Order/GroupWithZero/Canonical.lean,Mathlib/RingTheory/DedekindDomain/AdicValuation.lean |
2 |
2 |
['YaelDillies', 'github-actions'] |
nobody |
5-47329 5 days ago |
5-47329 5 days ago |
5-57120 5 days |
26448 |
YaelDillies author:YaelDillies |
refactor: simplify `(f₁ ⊗ₘ f₂) ≫ (g₁ ⊗ₘ g₂)` to `(f₁ ≫ g₁) ⊗ₘ (f₂ ≫ g₂)` |
... instead of the other way around. This is motivated by the fact that homs happening "in parallel" is a non-concept (time along a branch can always be reparametrised), while homs happening "in series" is a well-defined concept. One should not simp the well-defined concept into the non-concept but instead the other way around.
This is also motivated by the advent of the `mon_tauto` simp set in #26057.
From Toric
---
[](https://gitpod.io/from-referrer/)
|
toric
t-category-theory
|
115/119 |
Mathlib/Algebra/Category/ModuleCat/Monoidal/Basic.lean,Mathlib/Algebra/Category/ModuleCat/Presheaf/Monoidal.lean,Mathlib/CategoryTheory/Bicategory/End.lean,Mathlib/CategoryTheory/Dialectica/Monoidal.lean,Mathlib/CategoryTheory/Enriched/Basic.lean,Mathlib/CategoryTheory/Enriched/FunctorCategory.lean,Mathlib/CategoryTheory/GradedObject/Braiding.lean,Mathlib/CategoryTheory/GradedObject/Monoidal.lean,Mathlib/CategoryTheory/Localization/Monoidal.lean,Mathlib/CategoryTheory/Monoidal/Braided/Basic.lean,Mathlib/CategoryTheory/Monoidal/Braided/Reflection.lean,Mathlib/CategoryTheory/Monoidal/Cartesian/Basic.lean,Mathlib/CategoryTheory/Monoidal/Category.lean,Mathlib/CategoryTheory/Monoidal/Free/Basic.lean,Mathlib/CategoryTheory/Monoidal/Functor.lean,Mathlib/CategoryTheory/Monoidal/FunctorCategory.lean,Mathlib/CategoryTheory/Monoidal/Internal/Limits.lean,Mathlib/CategoryTheory/Monoidal/Limits.lean,Mathlib/CategoryTheory/Monoidal/Mon_.lean,Mathlib/CategoryTheory/Monoidal/NaturalTransformation.lean,Mathlib/CategoryTheory/Monoidal/Opposite.lean,Mathlib/CategoryTheory/Monoidal/Preadditive.lean,Mathlib/CategoryTheory/Monoidal/Transport.lean,Mathlib/CategoryTheory/Monoidal/Types/Coyoneda.lean |
24 |
12 |
['YaelDillies', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'robin-carlier', 'yuma-mizuno'] |
nobody |
5-46119 5 days ago |
5-47000 5 days ago |
21-1167 21 days |
27136 |
plp127 author:plp127 |
chore: mark argument explicit in `LinearOrder.toBiheytingAlgebra` |
Mark `α : Type*` explicit in `LinearOrder.toBiheytingAlgebra`. This matches better with what other similar reducible non-instances have.
---
[](https://gitpod.io/from-referrer/)
|
t-order |
17/14 |
Mathlib/Data/Fintype/Order.lean,Mathlib/Data/Nat/PartENat.lean,Mathlib/Order/CompleteLatticeIntervals.lean,Mathlib/Order/ConditionallyCompleteLattice/Basic.lean,Mathlib/Order/Fin/Basic.lean,Mathlib/Order/Heyting/Basic.lean |
6 |
1 |
['github-actions'] |
nobody |
5-45946 5 days ago |
5-46087 5 days ago |
5-46082 5 days |
27137 |
YaelDillies author:YaelDillies |
feat(CategoryTheory/Monoidal: an isomorphism of group objects is an isomorphim of the underlying objects |
From Toric
---
[](https://gitpod.io/from-referrer/)
|
toric
t-category-theory
|
12/0 |
Mathlib/CategoryTheory/Monoidal/CommGrp_.lean,Mathlib/CategoryTheory/Monoidal/CommMon_.lean,Mathlib/CategoryTheory/Monoidal/Grp_.lean,Mathlib/CategoryTheory/Monoidal/Mon_.lean |
4 |
1 |
['github-actions'] |
nobody |
5-45356 5 days ago |
5-45409 5 days ago |
5-45408 5 days |
27113 |
pechersky author:pechersky |
feat(RingTheory/SimpleRing/Principal): a commutative simple ring is a PID |
via `IsField` and new `IsField.isDomain`
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
41/2 |
Mathlib.lean,Mathlib/Algebra/Field/IsField.lean,Mathlib/RingTheory/PrincipalIdealDomain.lean,Mathlib/RingTheory/SimpleRing/Principal.lean |
4 |
4 |
['alreadydone', 'github-actions'] |
nobody |
5-43671 5 days ago |
5-85075 5 days ago |
5-85069 5 days |
26282 |
AntoineChambert-Loir author:AntoineChambert-Loir |
feat: a theorem of Jordan on primitive subgroups of the permutation group |
A theorem of Jordan on the primitive subgroups of a permutation group:
* if it contains a swap, it is equal to the permutation group,
* if it contains a 3-cycle, it contains the alternating group.
This PR continues the work from #24131.
- [x] depends on: #26281
- [x] depends on: #26280
- [x] depends on: #26279
Original PR: https://github.com/leanprover-community/mathlib4/pull/24131
[](https://gitpod.io/from-referrer/) |
large-import |
1084/183 |
Mathlib.lean,Mathlib/Data/Set/Card.lean,Mathlib/GroupTheory/GroupAction/Jordan.lean,Mathlib/GroupTheory/GroupAction/MultiplePrimitivity.lean,Mathlib/GroupTheory/GroupAction/MultipleTransitivity.lean,Mathlib/GroupTheory/GroupAction/Primitive.lean,Mathlib/GroupTheory/GroupAction/SubMulAction/OfFixingSubgroup.lean,Mathlib/GroupTheory/GroupAction/SubMulAction/OfStabilizer.lean,Mathlib/GroupTheory/Perm/Cycle/Type.lean,Mathlib/SetTheory/Cardinal/Embedding.lean |
10 |
n/a |
['AntoineChambert-Loir', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'tb65536'] |
nobody |
5-42736 5 days ago |
unknown |
unknown |
27118 |
Timeroot author:Timeroot |
feat(Matrix/Charpoly/Eigs): Roots of Matrix.charpoly are the eigenvalues. |
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebra
label:t-algebra$ |
58/0 |
Mathlib/LinearAlgebra/Matrix/Charpoly/Eigs.lean,scripts/noshake.json |
2 |
1 |
['github-actions'] |
nobody |
5-40129 5 days ago |
5-79630 5 days ago |
5-79673 5 days |
25910 |
themathqueen author:themathqueen |
feat(Algebra/Ring/Idempotent): subtraction lemmas for idempotents and star projections |
This allows us to use subtraction with idempotents and star projections.
For idempotents `p,q`, `q - p` is idempotent when `p * q = p = q * p`.
For star projections `p,q`, `q - p` is a star projection when either `p * q = p` or `q * p = p`. In a star-ordered ring, when `p * q = p` or `q * p = p` we get `p ≤ q`.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-algebra
label:t-algebra$ |
70/0 |
Mathlib/Algebra/Order/Star/Basic.lean,Mathlib/Algebra/Ring/Idempotent.lean,Mathlib/Algebra/Star/StarProjection.lean |
3 |
23 |
['github-actions', 'tb65536', 'themathqueen'] |
nobody |
5-33934 5 days ago |
19-81686 19 days ago |
22-29447 22 days |
25781 |
emilyriehl author:emilyriehl |
Feat(CategoryTheory): terminal categories with an application to hoFunctor |
Some preliminary API around terminal categories is developed with an application for the infinity-cosmos project: proving that the homotopy category functor preserves terminal objects. We also include proofs that `[0]` is terminal in the simplex category and `Δ[0]` is the terminal simplicial set.
Co-authored by [Robin Carlier](robin.carlier@ens-lyon.fr), [Jakob von Raumer](https://github.com/javra), [Adam Topaz](topaz@ualberta.ca), and [Zeyi Zhao](zzhao95@jh.edu).
---
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #25459.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/25459* |
infinity-cosmos
large-import
t-category-theory
|
185/2 |
Mathlib.lean,Mathlib/AlgebraicTopology/SimplexCategory/Basic.lean,Mathlib/AlgebraicTopology/SimplicialSet/HomotopyCat.lean,Mathlib/AlgebraicTopology/SimplicialSet/Monoidal.lean,Mathlib/CategoryTheory/Category/Cat/Terminal.lean,Mathlib/CategoryTheory/Category/ReflQuiv.lean,Mathlib/CategoryTheory/EssentiallySmall.lean,Mathlib/CategoryTheory/Quotient.lean |
8 |
27 |
['emilyriehl', 'github-actions', 'joelriou'] |
nobody |
5-32986 5 days ago |
7-26557 7 days ago |
20-27527 20 days |
27090 |
TerenceGitH author:TerenceGitH |
feat(Topology, Archive/Examples): Kuratowski's closure-complement theorem (incl. sharpness) |
This is the outcome of a course project at Heidelberg University: https://matematiflo.github.io/CompAssistedMath2025/
feat(Topology): Kuratowski's closure-complement theorem
"Topology/Kuratowski.lean" proves Kuratowski's closure-complement theorem, which says that if one repeatedly applies the closure and complement operators to a set in a topological space, at most 14 distinct sets can be obtained.
feat(Archive/Examples): sharpness of Kuratowski's closure-complement theorem:
"Examples/Kuratowski.lean" gives an example of a so-called "14-set" in ℝ, from which exactly 14 distinct sets can be obtained.
Co-authored-by: Luis Sand @luiis-sd
Co-authored-by: Leon Müller @leondieprobifi
Co-authored-by: Junyan Xu @alreadydone
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-topology
|
386/0 |
Archive.lean,Archive/Examples/Kuratowski.lean,Mathlib.lean,Mathlib/Topology/Kuratowski.lean |
4 |
5 |
['alreadydone', 'github-actions', 'wwylele'] |
nobody |
5-26337 5 days ago |
6-29860 6 days ago |
6-31202 6 days |
26122 |
chrisflav author:chrisflav |
refactor(CategoryTheory/CoproductDisjoint): generalize to indexed coproducts |
We replace the currently existing `CoproductDisjoint` by a predicate for a family of objects, indicating that the pairwise
pullbacks are disjoint and the coproduct inclusions are monomorphisms.
The old predicate is recovered as `BinaryCoproductDisjoint` as an `abbrev`.
We also replace `CoproductsDisjoint` by `CoproductsOfShapeDisjoint` and `BinaryCoproductsDisjoint`. We postpone
the TODO to show that if binary coproducts are disjoint and suitable coproducts exist, then all coproducts of suitable shape are disjoint.
Note that `CoproductDisjoint` changed its meaning, so no deprecation can be added. This should be fine, since it is a leaf file that is hopefully not much used downstream.
Zulip discussion: https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/.60MonoCoprod.60.20and.20.60DisjointCoproduct.60/with/524752624
---
[](https://gitpod.io/from-referrer/)
|
t-category-theory |
198/89 |
Mathlib/CategoryTheory/Limits/Shapes/DisjointCoproduct.lean |
1 |
1 |
['github-actions'] |
robin-carlier assignee:robin-carlier |
4-77132 4 days ago |
31-28853 1 month ago |
31-28835 31 days |
26415 |
thorimur author:thorimur |
feat: basic translations between `X →o Y` and `X ⥤ Y` |
Adds basic definitions translating between `X →o Y` and `X ⥤ Y` where `X` and `Y` are regarded as `Preorder` categories.
---
[](https://gitpod.io/from-referrer/)
|
t-category-theory |
53/14 |
Mathlib/CategoryTheory/Category/Preorder.lean |
1 |
2 |
['github-actions', 'thorimur'] |
robin-carlier assignee:robin-carlier |
4-77124 4 days ago |
24-14004 24 days ago |
24-14344 24 days |
26663 |
joelriou author:joelriou |
feat(CategoryTheory/Abelian/SerreClass): left Bousfield localizations |
If `G : D ⥤ C` is an exact functor between abelian categories, with a fully faithful right adjoint `F`, then `G` identifies `C` to the localization of `D` with respect to the class of morphisms `G.kernel.isoModSerre`, i.e. `D` is the localization of `C` with respect to Serre class `G.kernel` consisting of the objects in `D` that are sent to a zero object by `G`. (We also translate this in terms of a left Bousfield localization.)
---
This PR continues the work from #22741.
Original PR: https://github.com/leanprover-community/mathlib4/pull/22741 |
t-category-theory |
89/2 |
Mathlib.lean,Mathlib/CategoryTheory/Abelian/SerreClass/Bousfield.lean,Mathlib/CategoryTheory/Abelian/SerreClass/MorphismProperty.lean,Mathlib/CategoryTheory/ObjectProperty/ContainsZero.lean |
4 |
1 |
['github-actions'] |
robin-carlier assignee:robin-carlier |
4-77119 4 days ago |
16-58910 16 days ago |
16-58929 16 days |
26169 |
joelriou author:joelriou |
feat(AlgebraicTopology/ModelCategory): a trick by Joyal |
In order to construct a model category, we may sometimes have basically proven all the axioms with the exception of the left lifting property of cofibrations with respect to trivial fibrations. A trick by Joyal allows to obtain this lifting property under suitable assumptions, namely that cofibrations are stable under composition and cobase change. (The dual statement is also formalized.)
This will be used in the formalization of the model category structure on topological spaces, simplicial sets, simplicial presheaves, etc.
---
- [x] depends on: #26166
This PR continues the work from #20224.
Original PR: https://github.com/leanprover-community/mathlib4/pull/20224 |
large-import
t-category-theory
|
100/0 |
Mathlib.lean,Mathlib/AlgebraicTopology/ModelCategory/JoyalTrick.lean,docs/references.bib |
3 |
4 |
['github-actions', 'joelriou', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
robin-carlier assignee:robin-carlier |
4-77107 4 days ago |
13-36970 13 days ago |
13-37003 13 days |
26972 |
joelriou author:joelriou |
feat(CategoryTheory): localization of quotient categories |
Under certain circumstances, we show that the localized category of a quotient category identifies to the localization of the original category.
---
[](https://gitpod.io/from-referrer/)
|
t-category-theory |
108/0 |
Mathlib.lean,Mathlib/CategoryTheory/Localization/LocalizerMorphism.lean,Mathlib/CategoryTheory/Localization/Predicate.lean,Mathlib/CategoryTheory/Localization/Quotient.lean |
4 |
2 |
['github-actions', 'joelriou'] |
robin-carlier assignee:robin-carlier |
4-72407 4 days ago |
9-45539 9 days ago |
9-45522 9 days |
22771 |
alreadydone author:alreadydone |
feat(Homotopy/Lifting): monodromy of covering maps and lifting criterion |
Definition 2.1 in https://ncatlab.org/nlab/show/monodromy.
Also:
+ Extract `FundamentalGroupoid.map (f : C(X, Y)) : FundamentalGroupoid X ⥤ FundamentalGroupoid Y` from `fundamentalGroupoidFunctor : TopCat ⥤ CategoryTheory.Grpd`
+ Define `FundamentalGroup.map (f : C(X, Y)) (x : X) : FundamentalGroup X x →* FundamentalGroup Y (f x)` and `mapOfEq : FundamentalGroup X x →* FundamentalGroup Y y` that takes an assumption `f x = y`.
+ Redefine `FundamentalGroup` to be `End` rather than `Aut`: since `FundamentalGroupoid` is a groupoid, `End` already has a group structure.
+ Golf within the file FundamentalGroupoid/Basic.
+ Generalize `toArrow` up to `fromPath` in `FundamentalGroupoid/FundamentalGroup` from `X : TopCat` to `[TopologicalSpace X]`.
Also golfs some proofs and redefines
---
- [x] depends on: #22649
[](https://gitpod.io/from-referrer/)
|
t-topology |
193/147 |
Mathlib/AlgebraicTopology/FundamentalGroupoid/Basic.lean,Mathlib/AlgebraicTopology/FundamentalGroupoid/FundamentalGroup.lean,Mathlib/AlgebraicTopology/FundamentalGroupoid/InducedMaps.lean,Mathlib/AlgebraicTopology/FundamentalGroupoid/SimplyConnected.lean,Mathlib/CategoryTheory/Groupoid.lean,Mathlib/Topology/Covering.lean,Mathlib/Topology/Homotopy/HomotopyGroup.lean,Mathlib/Topology/Homotopy/Lifting.lean,Mathlib/Topology/Homotopy/Product.lean |
9 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
PatrickMassot assignee:PatrickMassot |
4-64144 4 days ago |
14-30535 14 days ago |
122-10064 122 days |
26655 |
Rida-Hamadani author:Rida-Hamadani |
feat(SimpleGraph): sub-walks |
defines (contiguous) subwalks and provides lemmas about them.
Co-authored-by: Kyle Miller
Co-authored-by: Vlad Tsyrklevich
---
[](https://gitpod.io/from-referrer/)
|
t-combinatorics |
176/0 |
Mathlib/Combinatorics/SimpleGraph/Paths.lean,Mathlib/Combinatorics/SimpleGraph/Walk.lean,Mathlib/Data/List/Infix.lean |
3 |
20 |
['Rida-Hamadani', 'github-actions', 'jt496', 'kmill', 'vlad902'] |
nobody |
4-55511 4 days ago |
16-73014 16 days ago |
16-73065 16 days |
27087 |
staroperator author:staroperator |
feat(Data/Set): add `sep_subset_setOf` |
which is the counterpart of `sep_subset` for use in term mode.
---
[](https://gitpod.io/from-referrer/)
|
t-data
new-contributor
easy
|
3/0 |
Mathlib/Data/Set/Basic.lean |
1 |
1 |
['github-actions'] |
nobody |
4-46859 4 days ago |
6-38419 6 days ago |
6-38463 6 days |
27088 |
staroperator author:staroperator |
feat(Algebra/Order/Sub): add `map_tsub_of_le` |
An `AddHom` keeps ordered subtraction in canonically ordered monoids. This is a simple corollary of `tsub_add_cancel_of_le`.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-algebra
label:t-algebra$ |
8/1 |
Mathlib/Algebra/Order/Sub/Unbundled/Hom.lean |
1 |
1 |
['github-actions'] |
nobody |
4-46853 4 days ago |
6-37815 6 days ago |
6-37861 6 days |
27163 |
pechersky author:pechersky |
feat(Topology/ValuativeRel): of and to basis of compatible valuations |
---
[](https://gitpod.io/from-referrer/)
|
|
109/5 |
Mathlib/RingTheory/Valuation/ValuativeRel.lean,Mathlib/Topology/Algebra/Valued/ValuativeRel.lean |
2 |
1 |
['github-actions'] |
nobody |
4-46065 4 days ago |
4-49064 4 days ago |
4-49046 4 days |
11563 |
YaelDillies author:YaelDillies |
feat: `∑ i ∈ s with hi : p i, f i hi` syntax for big operators |
Define new notation for `Finset.sum`/`Finset.prod`. `∑ i ∈ s with hi : p i, f i hi` now is notation for `∑ i : s.filter p, f i.1 (mem_filter.1 i.2).2`.
---
- [x] depends on: #6795
Other notations we could have are
* `∑ hi : i ∈ s, f i hi` as notation for `∑ i : s, f i.1 i.2`
* `∑ hi : i ∈ s with p i, f i hi` as notation for `∑ i : s.filter p, f i.1 (mem_filter.1 i.2).1`
* `∑ hi : i ∈ s with hpi : p i, f i hi hpi` as notation for `∑ i : s.filter p, f i.1 (mem_filter.1 i.2).1 (mem_filter.1 i.2).2`
but Eric seems mildly unhappy about them.
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-meta
label:t-algebra$ |
27/18 |
Mathlib/Algebra/BigOperators/Group/Finset/Defs.lean |
1 |
28 |
['YaelDillies', 'b-mehta', 'eric-wieser', 'github-actions', 'kbuzzard', 'kmill', 'leanprover-community-bot-assistant', 'leanprover-community-mathlib4-bot'] |
kmill assignee:kmill |
4-43820 4 days ago |
4-43844 4 days ago |
166-31801 166 days |
25042 |
alreadydone author:alreadydone |
feat(Topology): restriction/extension of Trivialization and composition with Homeomorph |
---
- [x] depends on: #25041
[](https://gitpod.io/from-referrer/)
|
t-topology |
148/2 |
Mathlib/Topology/FiberBundle/Trivialization.lean,Mathlib/Topology/Maps/Basic.lean |
2 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
4-43338 4 days ago |
4-63536 4 days ago |
60-46804 60 days |
27035 |
faenuccio author:faenuccio |
chore(IsManifold/Basic): replace continuity by aesop |
---
[](https://gitpod.io/from-referrer/)
|
t-differential-geometry
easy
|
5/5 |
Mathlib/Geometry/Manifold/IsManifold/Basic.lean |
1 |
3 |
['faenuccio', 'fpvandoorn', 'github-actions'] |
nobody |
4-43027 4 days ago |
7-42476 7 days ago |
7-45363 7 days |
9915 |
eric-wieser author:eric-wieser |
refactor: Add norm_num machinery for NNRat |
This splits the previous `isRat` primitive into `isNNRat` and `isNegNNRat`, where only the latter carries around a `DivisionRing` instance.
This means that `norm_num` works on `NNReal` and `NNRat`.
Co-authored-by: Aaron Liu
---
- [x] depends on: #9951
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-meta
label:t-algebra$ |
758/237 |
Mathlib/Analysis/SpecialFunctions/Log/Basic.lean,Mathlib/Analysis/SpecialFunctions/Pow/Real.lean,Mathlib/Data/Rat/Floor.lean,Mathlib/Tactic/NormNum/Basic.lean,Mathlib/Tactic/NormNum/BigOperators.lean,Mathlib/Tactic/NormNum/Eq.lean,Mathlib/Tactic/NormNum/Ineq.lean,Mathlib/Tactic/NormNum/Inv.lean,Mathlib/Tactic/NormNum/Irrational.lean,Mathlib/Tactic/NormNum/OfScientific.lean,Mathlib/Tactic/NormNum/Pow.lean,Mathlib/Tactic/NormNum/RealSqrt.lean,Mathlib/Tactic/NormNum/Result.lean,Mathlib/Tactic/Positivity/Core.lean,Mathlib/Tactic/Ring/Basic.lean,Mathlib/Tactic/Ring/RingNF.lean,MathlibTest/norm_num.lean,MathlibTest/norm_num_ext.lean,MathlibTest/ring.lean,scripts/nolints.json |
20 |
8 |
['eric-wieser', 'github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'plp127'] |
nobody |
4-35399 4 days ago |
6-41183 6 days ago |
16-40568 16 days |
27149 |
euprunin author:euprunin |
feat: slightly reduce the verbosity of `lake cache exe get` |
Along with reducing distracting verbosity, this change also addresses the confusing, seemingly contradictory output pair:
```
Downloaded: 6951 file(s) [attempted 6951/6951 = 100%] (100% success)
No files to download
```
Pre:
```
% lake exe cache get
Current branch: master
Using cache from origin: github-username/mathlib4
Attempting to download 6951 file(s) from leanprover-community/mathlib4 cache
Downloaded: 6951 file(s) [attempted 6951/6951 = 100%] (100% success)
No files to download
Decompressing 6951 file(s)
Unpacked in 546 ms
Completed successfully!
% lake exe cache get
Current branch: master
Using cache from origin: github-username/mathlib4
No files to download
No files to download
Decompressing 6951 file(s)
Unpacked in 320 ms
Completed successfully!
%
```
Post:
```
% lake exe cache get
Current branch: master
Using cache from origin: github-username/mathlib4
Attempting to download 6951 file(s) from leanprover-community/mathlib4 cache
Downloaded: 6951 file(s) [attempted 6951/6951 = 100%] (100% success)
Decompressing 6951 file(s)
% lake exe cache get
Current branch: master
Using cache from origin: github-username/mathlib4
Decompressing 6951 file(s)
%
```
Fixes #27038. Note that the download progress output is kept unchanged. |
|
0/4 |
Cache/IO.lean,Cache/Requests.lean |
2 |
2 |
['euprunin', 'github-actions'] |
nobody |
4-26868 4 days ago |
4-79342 4 days ago |
4-79324 4 days |
26726 |
euprunin author:euprunin |
chore: golf Algebra/ using `grind` |
|
t-algebra label:t-algebra$ |
58/160 |
Mathlib/Algebra/BigOperators/Group/Finset/Piecewise.lean,Mathlib/Algebra/BigOperators/Group/List/Lemmas.lean,Mathlib/Algebra/ContinuedFractions/Computation/CorrectnessTerminating.lean,Mathlib/Algebra/ContinuedFractions/ConvergentsEquiv.lean,Mathlib/Algebra/ContinuedFractions/Determinant.lean,Mathlib/Algebra/GeomSum.lean,Mathlib/Algebra/Group/UniqueProds/Basic.lean,Mathlib/Algebra/Homology/HomotopyCategory/HomComplex.lean,Mathlib/Algebra/Homology/TotalComplexShift.lean,Mathlib/Algebra/IsPrimePow.lean,Mathlib/Algebra/Module/Submodule/Range.lean,Mathlib/Algebra/MonoidAlgebra/Defs.lean,Mathlib/Algebra/MvPolynomial/CommRing.lean,Mathlib/Algebra/MvPolynomial/Degrees.lean,Mathlib/Algebra/MvPolynomial/Variables.lean,Mathlib/Algebra/Order/Antidiag/Nat.lean,Mathlib/Algebra/Order/BigOperators/Group/List.lean,Mathlib/Algebra/Order/BigOperators/GroupWithZero/List.lean,Mathlib/Algebra/Order/CompleteField.lean,Mathlib/Algebra/Polynomial/Coeff.lean,Mathlib/Algebra/Polynomial/Div.lean,Mathlib/Algebra/Polynomial/HasseDeriv.lean,Mathlib/Algebra/Polynomial/Module/Basic.lean,Mathlib/Algebra/Polynomial/UnitTrinomial.lean,Mathlib/Algebra/QuadraticDiscriminant.lean,Mathlib/Algebra/QuaternionBasis.lean,Mathlib/Algebra/TrivSqZeroExt.lean |
27 |
11 |
['github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'leanprover-community-mathlib4-bot'] |
nobody |
4-19018 4 days ago |
4-19018 4 days ago |
15-71223 15 days |
27152 |
xroblot author:xroblot |
feat(RingTheory/Ideal): prove transitivity for the relative norm |
---
- [x] depends on: #26070
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
149/15 |
Mathlib/Algebra/Algebra/Tower.lean,Mathlib/RingTheory/DedekindDomain/Ideal.lean,Mathlib/RingTheory/Ideal/Norm/RelNorm.lean,Mathlib/RingTheory/Ideal/Operations.lean,Mathlib/RingTheory/IntegralClosure/IntegralRestrict.lean,Mathlib/RingTheory/Localization/AtPrime.lean,Mathlib/RingTheory/Localization/FractionRing.lean |
7 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
riccardobrasca assignee:riccardobrasca |
4-18764 4 days ago |
4-18771 4 days ago |
4-29719 4 days |
27072 |
eric-wieser author:eric-wieser |
feat(Data/Matrix): more lemmas about `Matrix.vecMulVec` |
Inspired by [#new members > Is this a reasonable formalization? @ 💬](https://leanprover.zulipchat.com/#narrow/channel/113489-new-members/topic/Is.20this.20a.20reasonable.20formalization.3F/near/528412531).
---
[](https://gitpod.io/from-referrer/)
|
t-data |
66/0 |
Mathlib/Data/Matrix/ConjTranspose.lean,Mathlib/Data/Matrix/Mul.lean |
2 |
1 |
['github-actions'] |
nobody |
4-16993 4 days ago |
6-51534 6 days ago |
6-51575 6 days |
26644 |
kckennylau author:kckennylau |
feat(SetTheory/ZFC): Define the language of sets and state the ZFC axioms |
---
[](https://gitpod.io/from-referrer/)
|
t-set-theory |
381/0 |
Mathlib.lean,Mathlib/SetTheory/ZFC/Axioms.lean,docs/references.bib |
3 |
45 |
['github-actions', 'kckennylau', 'staroperator', 'vihdzp'] |
nobody |
4-9289 4 days ago |
17-17443 17 days ago |
17-17491 17 days |
27159 |
Parcly-Taxel author:Parcly-Taxel |
feat: IMO 1997 Q3 |
|
IMO |
129/0 |
Archive.lean,Archive/Imo/Imo1997Q3.lean |
2 |
5 |
['Parcly-Taxel', 'eric-wieser', 'github-actions'] |
nobody |
4-6760 4 days ago |
4-53855 4 days ago |
4-53843 4 days |
25770 |
Parcly-Taxel author:Parcly-Taxel |
chore: fix more induction/recursor branch names |
These were found using the regex `\| h. =>` and `def.*rec.*\(h. :`. |
tech debt |
134/115 |
Mathlib/Analysis/Convolution.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/Data/Fin/Tuple/Basic.lean,Mathlib/Data/Fin/Tuple/NatAntidiagonal.lean,Mathlib/Data/Nat/Factorization/Induction.lean,Mathlib/Data/Seq/Computation.lean,Mathlib/Data/Set/Card.lean,Mathlib/Data/WSeq/Basic.lean,Mathlib/FieldTheory/KummerExtension.lean,Mathlib/Logic/Function/Iterate.lean,Mathlib/NumberTheory/ArithmeticFunction.lean,Mathlib/NumberTheory/SumFourSquares.lean,Mathlib/NumberTheory/SumTwoSquares.lean,Mathlib/Order/SuccPred/Archimedean.lean,Mathlib/Order/Synonym.lean |
15 |
11 |
['Parcly-Taxel', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant'] |
nobody |
4-6656 4 days ago |
13-10719 13 days ago |
35-79507 35 days |
27160 |
kebekus author:kebekus |
feat: describe posLog in terms of circle averages |
If `a` is any complex number of norm one, establish by direct computation that the circle average `circleAverage (log ‖· - a‖) 0 1` vanishes.
As soon as the mean value theorem for harmonic functions becomes available, this result will be extended to arbitrary complex numbers `a`, showing that the circle average equals the positive part of the logarithm, `circleAverage (log ‖· - a‖) 0 1 = log⁺ ‖a‖`. This result, in turn, is a major ingredient in the proof of Jensen's formula in complex analysis.
---
[](https://gitpod.io/from-referrer/)
|
t-analysis |
98/0 |
Mathlib.lean,Mathlib/Analysis/SpecialFunctions/Integrals/PosLogEqCircleAverage.lean |
2 |
1 |
['github-actions'] |
nobody |
3-84147 3 days ago |
4-53249 4 days ago |
4-53296 4 days |
27178 |
artie2000 author:artie2000 |
feat(Algebra/Order/Ring): make `IsOrderedRing.toStrictOrderedRing` an instance |
Requiring `IsStrictOrderedRing` on a `Field` is a footgun (the current instances come from a find and replace on `LinearOrderedField`). Weakening typeclasses can incur a performance hit so will be done where appropriate in future PRs.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
1/1 |
Mathlib/Algebra/Order/Ring/Defs.lean |
1 |
4 |
['YaelDillies', 'github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot'] |
nobody |
3-75633 3 days ago |
4-17442 4 days ago |
4-30128 4 days |
26738 |
javra author:javra |
feat(AlgebraicToplogy/SimplexCategory): add notation for faces and degeneracies general truncated simplex categories |
---
[](https://gitpod.io/from-referrer/)
|
infinity-cosmos
t-topology
t-category-theory
|
41/29 |
Mathlib/AlgebraicTopology/SimplexCategory/Truncated.lean,Mathlib/AlgebraicTopology/SimplicialSet/HomotopyCat.lean |
2 |
3 |
['emilyriehl', 'github-actions', 'leanprover-community-bot-assistant'] |
nobody |
3-66984 3 days ago |
4-24328 4 days ago |
11-62829 11 days |
27166 |
joelriou author:joelriou |
feat(AlgebraicTopology): the functor `II : SimplexCategory ⥤ SimplexCategoryᵒᵖ` by Gabriel and Zisman |
In this file, we construct a cosimplicial object `SimplexCategory.II` in `SimplexCategoryᵒᵖ`, i.e. a functor `SimplexCategory ⥤ SimplexCategoryᵒᵖ`. If we identify `SimplexCategory` with the category of finite nonempty linearly ordered types, this functor could be interpreted as the contravariant functor which sends a finite nonempty linearly ordered type `T` to `T →o Fin 2`; in particular, it sends `Fin (n + 1)` to a linearly ordered type which is isomorphic to `Fin (n + 2)`. As a result, we define `SimplexCategory.II` as a functor which sends `⦋n⦌` to `⦋n + 1⦌`: on morphisms, it sends faces to degeneracies and vice versa.
(I plan to use this in order to show that the topological realization from simplicial sets to `TopCat` preserves finite limits, following the proof by Gabriel and Zisman.)
---
Suggestions for a better (short) name are welcome. `II` is the name given is the original source.
- [x] depends on: #27153
[](https://gitpod.io/from-referrer/)
|
t-category-theory |
258/0 |
Mathlib.lean,Mathlib/AlgebraicTopology/SimplicialObject/II.lean |
2 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
3-66931 3 days ago |
3-76772 3 days ago |
3-76763 3 days |
27194 |
YaelDillies author:YaelDillies |
feat: a finite monoid algebra is a finite module |
From Toric
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
28/1 |
Mathlib/RingTheory/Finiteness/Finsupp.lean |
1 |
2 |
['YaelDillies', 'eric-wieser', 'github-actions'] |
nobody |
3-64248 3 days ago |
3-72142 3 days ago |
3-72203 3 days |
27200 |
rotarc75 author:rotarc75 |
feat(RingTheory/Ideal): oka predicates over ideals |
This PR introduces the notion of Oka predicates over the ideals of a ring. We usually speak of [Oka families](https://stacks.math.columbia.edu/tag/05K9) but predicates seemed more in line with mathlib's conventions.
Currently this notions isn't used anywhere but we plan to make an other PR that proves that is all prime ideals of a ring are finitely generated, then this ring is Noetherian. We can also use Oka predicates to simplify the existing proof of [`IsPrincipalIdealRing.of_prime`](https://leanprover-community.github.io/mathlib4_docs/Mathlib/RingTheory/PrincipalIdealDomainOfPrime.html#IsPrincipalIdealRing.of_prime).
Co-authored-by: Anthony Fernandes
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-algebra
label:t-algebra$ |
53/0 |
Mathlib.lean,Mathlib/RingTheory/Ideal/Oka.lean |
2 |
1 |
['github-actions'] |
nobody |
3-62632 3 days ago |
3-62632 3 days ago |
3-63531 3 days |
27174 |
ADedecker author:ADedecker |
chore(OreLocalization): generalize some results from rings to monoids with zeros |
---
My motivation is getting a more conceptual construction of [ValuativeRel.ValueGroupWithZero](https://leanprover-community.github.io/mathlib4_docs/Mathlib/RingTheory/Valuation/ValuativeRel.html#ValuativeRel.ValueGroupWithZero), but I think this is of independent interest.
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
104/65 |
Mathlib.lean,Mathlib/RingTheory/OreLocalization/Basic.lean,Mathlib/RingTheory/OreLocalization/NonZeroDivisors.lean,Mathlib/RingTheory/OreLocalization/Ring.lean |
4 |
1 |
['github-actions'] |
nobody |
3-60673 3 days ago |
4-39297 4 days ago |
4-39350 4 days |
26931 |
javra author:javra |
feat(CategoryTheory/Enriched): `V`-enriched isomorphisms |
Defines isomorphisms in `V`-enriched categories and relate them to ordinary isomorphisms in the case of ordinary enriched categories.
---
[](https://gitpod.io/from-referrer/)
|
infinity-cosmos
t-category-theory
|
246/13 |
Mathlib.lean,Mathlib/CategoryTheory/Enriched/Basic.lean,Mathlib/CategoryTheory/Enriched/Iso.lean,Mathlib/CategoryTheory/Enriched/Opposite.lean,Mathlib/CategoryTheory/Enriched/Ordinary/Basic.lean,Mathlib/CategoryTheory/Enriched/Ordinary/Iso.lean |
6 |
8 |
['emilyriehl', 'github-actions', 'javra', 'mckoen'] |
nobody |
3-57407 3 days ago |
10-58671 10 days ago |
10-59656 10 days |
27169 |
YaelDillies author:YaelDillies |
chore(GroupTheory/FreeAbelianGroup): do not import cardinals |
Move the `Fintype` and `Cardinal` material from `GroupTheory.Coset.Basic` to `GroupTheory.Coset.Card`. That was just misplaced.
Split `GroupTheory.Abelianization` into:
* more material in `GroupTheory.Commutator.Basic` and `GroupTheory.Commutator.Finite` that was just misplaced
* `GroupTheory.Abelianization.Defs` for the definition of the abelianisation
* `GroupTheory.Abelianization.Finite` for the finiteness of the abelianisation of a finite group
---
[](https://gitpod.io/from-referrer/)
|
file-removed
large-import
|
439/411 |
Mathlib.lean,Mathlib/Algebra/Category/Grp/Adjunctions.lean,Mathlib/Algebra/Colimit/Ring.lean,Mathlib/Algebra/FreeAbelianGroup/Finsupp.lean,Mathlib/Algebra/FreeAbelianGroup/UniqueSums.lean,Mathlib/GroupTheory/Abelianization.lean,Mathlib/GroupTheory/Abelianization/Defs.lean,Mathlib/GroupTheory/Abelianization/Finite.lean,Mathlib/GroupTheory/Commutator/Basic.lean,Mathlib/GroupTheory/Commutator/Finite.lean,Mathlib/GroupTheory/CommutingProbability.lean,Mathlib/GroupTheory/Coset/Basic.lean,Mathlib/GroupTheory/Coset/Card.lean,Mathlib/GroupTheory/FreeAbelianGroup.lean,Mathlib/GroupTheory/GroupAction/Iwasawa.lean,Mathlib/GroupTheory/GroupAction/Quotient.lean,Mathlib/GroupTheory/Schreier.lean,Mathlib/GroupTheory/Solvable.lean,Mathlib/GroupTheory/SpecificGroups/Alternating/Centralizer.lean,Mathlib/GroupTheory/SpecificGroups/ZGroup.lean,Mathlib/RepresentationTheory/Homological/GroupHomology/LowDegree.lean,Mathlib/RingTheory/FreeCommRing.lean,Mathlib/RingTheory/FreeRing.lean,Mathlib/RingTheory/MvPolynomial/FreeCommRing.lean,Mathlib/SetTheory/Cardinal/Free.lean,Mathlib/Topology/Algebra/Group/TopologicalAbelianization.lean |
26 |
1 |
['github-actions'] |
nobody |
3-53345 3 days ago |
4-44044 4 days ago |
4-44107 4 days |
27207 |
pechersky author:pechersky |
feat(Topology/WithVal): ValuativeRel (WithVal v) |
with a helper valuation defined that does not pierce defeq
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-topology
label:t-algebra$ |
23/0 |
Mathlib/Topology/Algebra/Valued/WithVal.lean |
1 |
1 |
['github-actions'] |
nobody |
3-52554 3 days ago |
3-52555 3 days ago |
3-52869 3 days |
27210 |
YaelDillies author:YaelDillies |
feat: `MonoidHom.toHomUnits` is a monoid hom |
From Toric
---
[](https://gitpod.io/from-referrer/)
|
toric
large-import
t-algebra
label:t-algebra$ |
21/4 |
Mathlib/Algebra/Group/Units/Hom.lean |
1 |
1 |
['github-actions'] |
nobody |
3-51141 3 days ago |
3-51492 3 days ago |
3-51635 3 days |
27199 |
YaelDillies author:YaelDillies |
feat(MonoidAlgebra): miscellaneous basic lemmas |
From Toric
---
[](https://gitpod.io/from-referrer/)
|
toric
t-algebra
label:t-algebra$ |
50/9 |
Counterexamples/ZeroDivisorsInAddMonoidAlgebras.lean,Mathlib/Algebra/MonoidAlgebra/Defs.lean,Mathlib/Algebra/MvPolynomial/Degrees.lean,scripts/nolints.json |
4 |
1 |
['github-actions'] |
nobody |
3-50430 3 days ago |
3-63400 3 days ago |
3-63621 3 days |
27099 |
staroperator author:staroperator |
feat(ModelTheory): the language of Presburger Arithmetic |
This PR introduces the first-order language of [Presburger Arithmetic](https://en.wikipedia.org/wiki/Presburger_arithmetic). It has not defined the theory of Presburger Arithmetic yet (left as TODO), but is enough to prove some definability results (#27100).
---
[](https://gitpod.io/from-referrer/)
|
t-logic |
125/0 |
Mathlib.lean,Mathlib/ModelTheory/Arithmetic/Presburger/Basic.lean |
2 |
19 |
['YaelDillies', 'github-actions', 'staroperator'] |
nobody |
3-50200 3 days ago |
4-5847 4 days ago |
6-1448 6 days |
26679 |
robin-carlier author:robin-carlier |
feat(CategoryTheory/Limits/Shapes/Pullback/Categorical): 2-functoriality of `CatCommSqOver` |
This PR uses the notion of categorical cospan transforms from #26412 and its bicategory-like notations from #26447 to provide API for 2-functoriality of the construction `CatCommSqOver F G X`. We show that `ψ : CatCospanTransform F G F' G'` defines a functor `CatCommSqOver F G X ⥤ CatCommSqOver F' G' X`, and that a functor `U : X ⥤ Y` induces a functor `CatCommSqOver F G Y ⥤ CatCommSqOver F G X` via precomposition. We give the battery of lemma that shows that these constructions are components of a `Cat`-valued "bipseudofunctor", although we cannot state it this way to keep things unbundled and universe polymorphic.
---
- [x] depends on: #26447
I apologize in advance, for this one is very boring. As usual, the higher order lemmas are found by aesop_cat and are not marked simp, but I still want to state these explicitly so that in case automation goes wrong, "manual formal bicategory manipulations" remain an option.
A design choice was made here. Instead of stating this kind of functoriality for the categorical pullback itself, I chose to state everything in terms of `CatCommSqOver`, i.e in terms of the pseudofunctorial construction corepresented by the categorical pullback. The rationale here is that while we could have done everything only at the level of the categorical pullback itself, I believe this design will allow for easier manipulations of categorical pullback *squares*.
Actual bifunctoriality of the categorical pullback (and thus equivalence invariance, which is the key point of the notion compared to the strict pullback) will be in future PRs.
[](https://gitpod.io/from-referrer/)
|
t-category-theory |
408/1 |
Mathlib/CategoryTheory/Limits/Shapes/Pullback/Categorical/Basic.lean |
1 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
3-45000 3 days ago |
4-60077 4 days ago |
4-60077 4 days |
26875 |
michaellee94 author:michaellee94 |
feat(Manifold/PartitionOfUnity): existence of global C^n smooth section for nontrivial bundles |
Add existence of global C^n smooth section for nontrivial bundles
---
- [x] depends on: #26671
[](https://gitpod.io/from-referrer/) |
t-differential-geometry |
121/14 |
Mathlib/Geometry/Manifold/PartitionOfUnity.lean |
1 |
6 |
['github-actions', 'grunweg', 'mathlib4-dependent-issues-bot', 'michaellee94'] |
nobody |
3-41411 3 days ago |
9-39233 9 days ago |
9-53904 9 days |
27182 |
eric-wieser author:eric-wieser |
feat: add bundled versions of `Equiv.cast` |
These are essentially the non-categorical versions of `eqToHom`.
These are helpful to state some functorial results about things like `DFinsupp.equivCongrLeft` (with the alternative being to use an evil triangle somewhere instead).
[#Is there code for X? > LinearEquiv.cast / AddEquiv.cast etc @ 💬](https://leanprover.zulipchat.com/#narrow/channel/217875-Is-there-code-for-X.3F/topic/LinearEquiv.2Ecast.20.2F.20AddEquiv.2Ecast.20etc/near/521390380)
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
31/0 |
Mathlib/Algebra/Algebra/Equiv.lean,Mathlib/Algebra/Group/Equiv/Defs.lean,Mathlib/Algebra/Module/Equiv/Defs.lean,Mathlib/Algebra/Ring/Equiv.lean |
4 |
3 |
['github-actions', 'pechersky', 'plp127'] |
nobody |
3-41320 3 days ago |
4-19883 4 days ago |
4-19925 4 days |
27192 |
RemyDegenne author:RemyDegenne |
feat: `covarianceBilin` lemmas |
Co-authored-by: Etienne Marion @EtienneC30
From the Brownian motion project.
---
[](https://gitpod.io/from-referrer/)
|
t-measure-probability |
33/4 |
Mathlib/Probability/Moments/CovarianceBilin.lean |
1 |
3 |
['EtienneC30', 'github-actions'] |
nobody |
3-38079 3 days ago |
3-38129 3 days ago |
3-65206 3 days |
26998 |
RemyDegenne author:RemyDegenne |
feat(Probability): covariance of sums and maps |
Variance and covariance of sums of random variables.
Covariance with respect to the map of a measure.
Co-authored-by: @EtienneC30
From the Brownian motion project.
---
[](https://gitpod.io/from-referrer/)
|
t-measure-probability |
157/1 |
Mathlib/MeasureTheory/Function/LpSeminorm/Defs.lean,Mathlib/Probability/Moments/Covariance.lean,Mathlib/Probability/Moments/Variance.lean |
3 |
7 |
['EtienneC30', 'github-actions'] |
nobody |
3-37997 3 days ago |
3-38065 3 days ago |
8-45180 8 days |
26914 |
quangvdao author:quangvdao |
feat(Data/PFunctor/Univariate): more definitions for univariate `PFunctor` |
This PR defines several basic definitions of `PFunctor`, including zero, one, constants, monomials, coproduct (sum), product, sigma, pi, tensor product, universe lifting, and equivalence.
We also add: (1) simple lemmas connecting the basic definitions, (2) an automatically derived ext lemma for `PFunctor` via `@[ext]` attribute
Some things I'm not clear on:
- I define `HAdd` and `HMul` instances for coproduct and product of poly functors having different universe levels. Should I also define `Add` and `Mul` instances for poly functors having the same universe level?
- Is it ok to define notation for tensor product, i.e. `@[inherit_doc] scoped infixr:80 " ⊗ " => tensor`? I'm worried it might clash with other notation.
- Need a double-check on the priority of notation.
Some future definitions to add:
- Various equivalences arising from arithmetic identities, e.g., `P + 0 ≃ₚ P`.
- Definitions of Lenses and Charts (each of them will be a file or even a folder)
- Exponential objects (corresponding to both `prod` and `tensor`)
---
[](https://gitpod.io/from-referrer/)
|
t-data |
183/5 |
Mathlib/Data/PFunctor/Univariate/Basic.lean |
1 |
10 |
['alexkeizer', 'eric-wieser', 'github-actions', 'quangvdao'] |
nobody |
3-24479 3 days ago |
11-12761 11 days ago |
11-12806 11 days |
27127 |
RemyDegenne author:RemyDegenne |
feat(Probability): 2 processes have same law iff same finite dimensional laws |
Co-authored-by: Jonas Bayer @TBUGTB
From the Brownian motion project.
---
[](https://gitpod.io/from-referrer/)
|
maintainer-merge
t-measure-probability
|
106/0 |
Mathlib.lean,Mathlib/Probability/Process/FiniteDimensionalLaws.lean |
2 |
5 |
['EtienneC30', 'github-actions'] |
nobody |
3-22828 3 days ago |
3-22828 3 days ago |
5-45801 5 days |
26921 |
grunweg author:grunweg |
feat: add mdifferentiable analogues of C^n metric lemmas |
---
- [ ] depends on: #26922
[](https://gitpod.io/from-referrer/)
|
t-differential-geometry |
56/0 |
Mathlib/Geometry/Manifold/VectorBundle/Riemannian.lean |
1 |
3 |
['github-actions', 'grunweg', 'mathlib4-dependent-issues-bot'] |
nobody |
3-18417 3 days ago |
3-36699 3 days ago |
3-37324 3 days |
25248 |
xcloudyunx author:xcloudyunx |
feat(Combinatorics/SimpleGraph): Add Subgraph.inclusion_edge_apply_coe and inclusion_edgeSet_apply_coe |
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-combinatorics
|
12/0 |
Mathlib/Combinatorics/SimpleGraph/Subgraph.lean |
1 |
3 |
['github-actions', 'pimotte', 'xcloudyunx'] |
nobody |
3-11261 3 days ago |
53-19695 1 month ago |
53-19747 53 days |
27226 |
xcloudyunx author:xcloudyunx |
feat(Combinatorics/SimpleGraph): Add Subgraph.inclusion_edge_apply_coe and inclusion_edgeSet_apply_coe |
This PR continues the work from #25248.
Original PR: https://github.com/leanprover-community/mathlib4/pull/25248 |
new-contributor
t-combinatorics
|
14/0 |
Mathlib/Combinatorics/SimpleGraph/Subgraph.lean |
1 |
1 |
['github-actions'] |
nobody |
3-9770 3 days ago |
3-11189 3 days ago |
3-11245 3 days |
27014 |
yuanyi-350 author:yuanyi-350 |
feat(GroupTheory/Perm/Fin): add Fin.cycleIcc and refactor cycleRange |
In this PR, I define the permutation `cycleIcc i j hij`, which is the cycle `(i i+1 .... j)` leaving `(0 ... i-1)` and `(j+1 ... n-1)` unchanged. In other words, it rotates elements in `[i, j]` one step to the right. Also I prove some properties of `cycleIcc i j hij` such as the fact that it is a cycle and its cycleType is `j - i`.
**This definition is used to prove the following result:**
```
theorem succAbove_comp_cycleIcc [NeZero n] (x : Fin (n + 1) → L) (i j : Fin (n + 1)) (eq : x i = x j) (lt : i < j)
x ∘ i.succAbove = x ∘ j.succAbove ∘ (cycleIcc hij)
```
More clearly, `x ∘ i.succAbove` and `x ∘ j.succAbove` are `Fin n → L` types. For example, when `n = 6, i = 2, j = 5` and `x i = x j`
```
x ∘ i.succAbove = (x 0, x 1, x 3, x 4, x 5, x 6)
x ∘ j.succAbove = (x 0, x 1, x 2, x 3, x 4, x 6)
```
We have
```
(x 0, x 1, x 3, x 4, x 5, x 6)
--(cycleIcc)--->(x 0, x 1, x 5, x 3, x 4, x 6) = (x 0, x 1, x 2, x 3, x 4, x 6)
```
---
Migrated from #24139
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
216/26 |
Mathlib/Algebra/Group/Fin/Basic.lean,Mathlib/Data/Fin/Basic.lean,Mathlib/Data/Fin/Embedding.lean,Mathlib/Data/Fin/SuccPred.lean,Mathlib/GroupTheory/Perm/Fin.lean |
5 |
55 |
['faenuccio', 'github-actions', 'mbkybky', 'yuanyi-350'] |
faenuccio assignee:faenuccio |
2-84805 2 days ago |
4-56886 4 days ago |
7-49637 7 days |
27224 |
alreadydone author:alreadydone |
fix(NonZeroDivisors): swap left and right |
Towards #22997:
+ Swap the definitions of `nonZeroDivisorsLeft` and `nonZeroDivisorsRight`, so as to conform to the convention in the literature (see https://en.wikipedia.org/wiki/Zero_divisor) and connects to mathlib's `IsLeftRegular` and `IsRightRegular` respectively without the presence of commutativity hypotheses.
+ Redefine `nonZeroDivisors` to be the intersection of `nonZeroDivisorsLeft` and `nonZeroDivisorsRight`, in analogy with `IsRegular`.
+ Swap `Commute.isNilpotent_mul_left/right(_iff)` as the names were also contrary to convention. (If the statement are left unchanged then the proofs need to be changed.)
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
255/131 |
Mathlib/Algebra/Group/Basic.lean,Mathlib/Algebra/GroupWithZero/NonZeroDivisors.lean,Mathlib/Algebra/Lie/Weights/Killing.lean,Mathlib/Algebra/Polynomial/AlgebraMap.lean,Mathlib/Algebra/Polynomial/Module/FiniteDimensional.lean,Mathlib/Algebra/Ring/NonZeroDivisors.lean,Mathlib/Dynamics/Newton.lean,Mathlib/FieldTheory/Laurent.lean,Mathlib/LinearAlgebra/Dimension/Torsion/Basic.lean,Mathlib/LinearAlgebra/Trace.lean,Mathlib/NumberTheory/ClassNumber/Finite.lean,Mathlib/NumberTheory/LegendreSymbol/AddCharacter.lean,Mathlib/RingTheory/Algebraic/Basic.lean,Mathlib/RingTheory/ClassGroup.lean,Mathlib/RingTheory/Ideal/MinimalPrime/Localization.lean,Mathlib/RingTheory/Ideal/Operations.lean,Mathlib/RingTheory/Localization/Cardinality.lean,Mathlib/RingTheory/Localization/Defs.lean,Mathlib/RingTheory/Localization/LocalizationLocalization.lean,Mathlib/RingTheory/MvPowerSeries/NoZeroDivisors.lean,Mathlib/RingTheory/Nilpotent/Basic.lean,Mathlib/RingTheory/Nilpotent/Defs.lean,Mathlib/RingTheory/Norm/Transitivity.lean,Mathlib/RingTheory/OreLocalization/Cardinality.lean,Mathlib/RingTheory/OreLocalization/Ring.lean,Mathlib/RingTheory/Polynomial/Nilpotent.lean,Mathlib/RingTheory/Polynomial/ScaleRoots.lean,Mathlib/RingTheory/PowerSeries/Substitution.lean,Mathlib/Topology/Sheaves/CommRingCat.lean |
29 |
3 |
['alreadydone', 'eric-wieser', 'github-actions'] |
nobody |
2-69188 2 days ago |
3-8747 3 days ago |
3-8747 3 days |
27184 |
JovanGerb author:JovanGerb |
chore(Order/Filter/Basic): write lemmas in point-free style |
This PR writes the congruence lemmas about filtered equality and about asymptotic equivalence in a point-free style. This is so that they can then be tagged with `@[gcongr]`. Some of the old versions have been kept with a `fun_` name.
And apparently the import size has decreased as a bonus :)
---
[](https://gitpod.io/from-referrer/)
|
t-order |
43/28 |
Mathlib/Analysis/Asymptotics/AsymptoticEquivalent.lean,Mathlib/Analysis/Normed/Ring/Units.lean,Mathlib/MeasureTheory/Function/LpSpace/Basic.lean,Mathlib/MeasureTheory/Function/LpSpace/Indicator.lean,Mathlib/MeasureTheory/Integral/Lebesgue/Add.lean,Mathlib/Order/Filter/Basic.lean,Mathlib/Order/Filter/Map.lean,Mathlib/Probability/Density.lean |
8 |
4 |
['JovanGerb', 'eric-wieser', 'github-actions'] |
nobody |
2-63225 2 days ago |
4-18937 4 days ago |
4-18981 4 days |
27092 |
smorel394 author:smorel394 |
feat(RingTheory.Finiteness.Finsupp, LinearAlgebra.DirectSum.Finite): a finite direct sum of finite modules is a finite module |
Prove that a finite direct sum of finite modules is a finite module.
There are instances both in the `DFinsupp` and `DirectSum` namespaces, to help type class inference find them.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
159/116 |
Mathlib.lean,Mathlib/Algebra/Module/FinitePresentation.lean,Mathlib/LinearAlgebra/Dimension/Finite.lean,Mathlib/LinearAlgebra/DirectSum/Finite.lean,Mathlib/RingTheory/Finiteness/ExactSequence.lean,Mathlib/RingTheory/Finiteness/Finsupp.lean,Mathlib/RingTheory/Finiteness/Ideal.lean,Mathlib/RingTheory/Noetherian/Basic.lean |
8 |
2 |
['github-actions', 'smorel394'] |
nobody |
2-58067 2 days ago |
4-52065 4 days ago |
6-29203 6 days |
27128 |
smorel394 author:smorel394 |
feat(CategoryTheory/Action/Basic, RepresentationTheory/FDRep): `Functor.mapAction F G` is fully faithful if `F` is |
Prove that, if a functor `F` is faithful (resp. fully faithful), then `F.mapAction G` is faithful (resp. full).
Apply this to the forgetful functor from `FGModuleCat k` to `ModuleCat k` to obtain that the forgetful functor from `FDRep k G` to `Rep k G` is fully faithful.
---
[](https://gitpod.io/from-referrer/)
|
t-category-theory |
24/0 |
Mathlib/CategoryTheory/Action/Basic.lean,Mathlib/RepresentationTheory/FDRep.lean |
2 |
1 |
['github-actions'] |
nobody |
2-58027 2 days ago |
5-56297 5 days ago |
5-56292 5 days |
27132 |
smorel394 author:smorel394 |
feat(CategoryTheory/Action/Limits): `F.mapAction G` preserves (co)limits |
Prove that `F.mapAction G : Action V G ⥤ Action W G` preserves (co)limits of some shape/size/etc if `F` preserves the same (co)limits and `V` has these (co)limits.
---
[](https://gitpod.io/from-referrer/)
|
t-category-theory |
82/6 |
Mathlib/CategoryTheory/Action/Limits.lean |
1 |
1 |
['github-actions'] |
nobody |
2-58020 2 days ago |
5-51588 5 days ago |
5-51586 5 days |
27154 |
smorel394 author:smorel394 |
feat(RingTheory/SimpleModule): a module over a semisimple ring is both injective and projective |
Prove that a module over a semisimple ring is both injective and projective. For the injectivity, this follows immediately from `IsSemisimpleModule.extension_property`. For the projectivity, we add a dual statement `IsSemisimpleModule.lifting_property` to `RingTheory.SimpleModule.Basic`. The actual `Module.Injective` and `Module.Projective` statements are in a separate file `RingTheory.SimpleModule.InjectiveProjective` to minimize imports in ``RingTheory.SimpleModule.Basic`.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
51/0 |
Mathlib.lean,Mathlib/RingTheory/SimpleModule/Basic.lean,Mathlib/RingTheory/SimpleModule/InjectiveProjective.lean |
3 |
1 |
['github-actions'] |
nobody |
2-57982 2 days ago |
4-64088 4 days ago |
4-64081 4 days |
26870 |
grunweg author:grunweg |
feat: mdifferentiableOn_section_of_mem_baseSet₀ |
From the path towards geodesics and the Levi-Civita connection.
Co-authored-by: Patrick Massot
---
- [x] depends on: #26866
[](https://gitpod.io/from-referrer/)
|
t-differential-geometry |
125/0 |
Mathlib/Geometry/Manifold/VectorBundle/MDifferentiable.lean |
1 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
2-53311 2 days ago |
2-53473 2 days ago |
2-53634 2 days |
27066 |
vasnesterov author:vasnesterov |
feat(Tactic/Order): frontend for `order` |
* Support `order [h1, h2]` and `order only [h1, h2]` syntax.
* Split conjunctions while extracting facts from the context. E.g. hypotheses in the form `A ∧ B` are converted into two facts `A` and `B`.
* Similarly, extract facts from existential quantifiers in the hypotheses.
---
- [x] depends on: #26354
[](https://gitpod.io/from-referrer/)
This PR continues the work from #22073.
Original PR: https://github.com/leanprover-community/mathlib4/pull/22073 |
t-meta |
92/29 |
Mathlib.lean,Mathlib/Tactic/Linarith/Frontend.lean,Mathlib/Tactic/Order.lean,Mathlib/Tactic/Order/CollectFacts.lean,Mathlib/Util/ElabWithoutMVars.lean,MathlibTest/order.lean |
6 |
22 |
['JovanGerb', 'github-actions', 'mathlib4-dependent-issues-bot', 'vasnesterov'] |
nobody |
2-49900 2 days ago |
6-67660 6 days ago |
6-67688 6 days |
27024 |
grunweg author:grunweg |
feat: Gram-Schmidt orthonormalisation for sections of a vector bundle |
Add a parametrised version of Gram-Schmidt, for sections of a topological vector bundle with a bundle metric.
This will be used to define orthonormal local frames.
From the path towards geodesics and the Levi-Civita connection.
Co-authored-by: Patrick Massot
---
- [x] depends on: #27023
[](https://gitpod.io/from-referrer/)
|
t-differential-geometry |
294/11 |
Mathlib.lean,Mathlib/Analysis/InnerProductSpace/GramSchmidtOrtho.lean,Mathlib/Geometry/Manifold/VectorBundle/GramSchmidtOrtho.lean,scripts/noshake.json |
4 |
59 |
['faenuccio', 'github-actions', 'grunweg', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
2-49121 2 days ago |
3-18821 3 days ago |
3-26371 3 days |
27021 |
grunweg author:grunweg |
feat: custom elaborators for differential geometry |
Add two sets of custom elaborators for differential geometry, to
- infer the model with corners in `MDifferentiable{WithinAt,At,On}` or `ContMDiff{WithinAt,At,On}` expressions from the local context, and provide shorter notation in that setting
- do the same for mfderiv: `mfderiv% f` is shorthand for `mfderiv I J f`; `mfderiv[s] f x` is short for `mfderivWithin I J f s`
- convert a fibre bundle section from a dependent section to a function into the total space, making working with differentiability of sections of fibre bundles less cumbersome
This was [discussed on zulip](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Differential.20geometry.20elaborators.20experiment/with/528035295), to overall broad consensus.
This code has substantial tests and has been tried in the branch in #26221 (uncovering minor issues, but not substantial ones). The implementation itself is of prototype quality and will be cleaned up in the future. Once it is more robust, more differential geometry files can be converted to use it.
Co-authored-by: Patrick Massot
-----------
I agree that merging not fully polished code is not ideal, but propose doing so for two reasons:
- the work in #26221 used these elaborators extensively (to test them). Reverting those changes, merging the code, only to re-apply them is not a good use of time. Merging this PR now enables merging the work in #26221 soon.
- the feature is clearly useful and not going away: in the files that use it, it works well already. Holding off on further adopting, but merging it now seems like a good compromise.
---
[](https://gitpod.io/from-referrer/)
|
t-differential-geometry
t-meta
|
782/0 |
Mathlib.lean,Mathlib/Geometry/Manifold/Elaborators.lean,Mathlib/Geometry/Manifold/Traces.lean,MathlibTest/DifferentialGeometry/Elaborators.lean,scripts/noshake.json |
5 |
4 |
['github-actions', 'grunweg', 'sgouezel'] |
nobody |
2-48420 2 days ago |
7-71349 7 days ago |
7-71422 7 days |
27006 |
zhikaip author:zhikaip |
refactor: crossProduct notation |
Replace `×₃` with `⨯` (`\X` or `\crossproduct`), and manually deprecate the old syntax.
See [#mathlib4 > Notation for crossProduct](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Notation.20for.20crossProduct/with/520119542)
---
[](https://gitpod.io/from-referrer/)
|
t-data
new-contributor
t-meta
|
37/22 |
Mathlib/Geometry/Euclidean/Angle/Unoriented/CrossProduct.lean,Mathlib/LinearAlgebra/CrossProduct.lean |
2 |
10 |
['eric-wieser', 'github-actions', 'j-loreaux', 'kmill'] |
nobody |
2-45551 2 days ago |
8-30987 8 days ago |
8-41012 8 days |
27229 |
WilliamCoram author:WilliamCoram |
feat(GroupTheory/DoubleCoset): multiple lemmas |
From FLT
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-algebra
label:t-algebra$ |
106/0 |
Mathlib/GroupTheory/DoubleCoset.lean |
1 |
1 |
['github-actions'] |
nobody |
2-45125 2 days ago |
2-45132 2 days ago |
2-45182 2 days |
27179 |
euprunin author:euprunin |
chore: golf `sub_convs_eq` using `field_simp` and `grind` |
|
t-algebra label:t-algebra$ |
2/10 |
Mathlib/Algebra/ContinuedFractions/Computation/Approximations.lean |
1 |
4 |
['euprunin', 'github-actions', 'grunweg'] |
nobody |
2-31352 2 days ago |
4-26277 4 days ago |
4-26321 4 days |
25905 |
mans0954 author:mans0954 |
feat(RingTheory/Polynomial/SmallDegreeVieta): polynomial versions of results in Algebra.QuadraticDiscriminant |
This PR continues the work from #25605.
Original PR: https://github.com/leanprover-community/mathlib4/pull/25605 |
t-algebra label:t-algebra$ |
73/8 |
Mathlib/RingTheory/Polynomial/SmallDegreeVieta.lean |
1 |
31 |
['github-actions', 'kckennylau', 'mans0954'] |
nobody |
2-29680 2 days ago |
34-57597 1 month ago |
34-57640 34 days |
26347 |
mans0954 author:mans0954 |
feature(Data/Finset/RangeDistance): abs_sub_lt_of_mem_finset_range |
This PR continues the work from #23161.
Original PR: https://github.com/leanprover-community/mathlib4/pull/23161 |
|
30/0 |
Mathlib.lean,Mathlib/Algebra/Order/Group/Unbundled/Abs.lean,Mathlib/Data/Finset/RangeDistance.lean |
3 |
2 |
['github-actions', 'mans0954'] |
nobody |
2-29471 2 days ago |
25-74503 25 days ago |
25-74485 25 days |
26350 |
mans0954 author:mans0954 |
feature(RingTheory/RootsOfUnity/Basic) : rootsOfUnity coercions |
This PR continues the work from #25215.
Original PR: https://github.com/leanprover-community/mathlib4/pull/25215 |
t-algebra label:t-algebra$ |
22/0 |
Mathlib/RingTheory/RootsOfUnity/Basic.lean |
1 |
2 |
['github-actions', 'mans0954'] |
nobody |
2-29429 2 days ago |
25-74077 25 days ago |
25-74119 25 days |
26836 |
mans0954 author:mans0954 |
feat(Order/Lattice): conditions for an equivalence relation to be a lattice congruence |
Define a structure asserting that a binary relation is a lattice congruence and provide sufficient and necessary conditions.
An application is given in #26983
---
- [x] depends on: #27219
[](https://gitpod.io/from-referrer/)
|
large-import
t-order
|
114/0 |
Mathlib/Order/Hom/Lattice.lean,Mathlib/Order/Lattice.lean,docs/references.bib |
3 |
20 |
['YaelDillies', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'mans0954', 'mathlib4-dependent-issues-bot'] |
nobody |
2-26161 2 days ago |
2-27682 2 days ago |
11-3816 11 days |
25907 |
mans0954 author:mans0954 |
Low order roots of unity |
This PR continues the work from #25470.
Original PR: https://github.com/leanprover-community/mathlib4/pull/25470 |
t-algebra label:t-algebra$ |
182/0 |
Mathlib/Algebra/CharP/Invertible.lean,Mathlib/RingTheory/RootsOfUnity/Complex.lean |
2 |
2 |
['github-actions', 'mans0954'] |
nobody |
2-25982 2 days ago |
34-57144 1 month ago |
34-57193 34 days |
27183 |
pechersky author:pechersky |
feat(RingTheory/ValuativeRel): IsRankLeOne when there is a compatible Zm0 or NNReal valuation |
and then provide it for Q_[p]
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-number-theory
label:t-algebra$ |
101/20 |
Mathlib/NumberTheory/Padics/ValuativeRel.lean,Mathlib/RingTheory/Valuation/ValuativeRel.lean |
2 |
12 |
['adamtopaz', 'github-actions', 'pechersky'] |
nobody |
2-24404 2 days ago |
2-24468 2 days ago |
3-19399 3 days |
27225 |
eric-wieser author:eric-wieser |
refactor(Tactic/Lift): deprecate the third with argument |
We already have a number of tactics where the clearing happens all the time, and you have to opt out with `id h`.
This also fixes a bug where `lift z to Nat with n hn this_is_unused` would silently ignore `this_is_unused`.
---
- [ ] depends on: #27223
[](https://gitpod.io/from-referrer/)
|
t-meta |
21/9 |
Mathlib/Tactic/Lift.lean,MathlibTest/lift.lean |
2 |
5 |
['JovanGerb', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'vihdzp'] |
nobody |
2-19276 2 days ago |
2-19299 2 days ago |
2-31779 2 days |
22782 |
alreadydone author:alreadydone |
feat(Topology): étalé space associated to a predicate on sections |
---
[](https://gitpod.io/from-referrer/)
|
t-topology |
886/160 |
Mathlib.lean,Mathlib/AlgebraicGeometry/ProjectiveSpectrum/StructureSheaf.lean,Mathlib/Data/Set/Operations.lean,Mathlib/Geometry/Manifold/Sheaf/Smooth.lean,Mathlib/Logic/Equiv/Basic.lean,Mathlib/Topology/EtaleSpace.lean,Mathlib/Topology/IsLocalHomeomorph.lean,Mathlib/Topology/Sheaves/LocalPredicate.lean,Mathlib/Topology/Sheaves/Sheafify.lean,Mathlib/Topology/Sheaves/Stalks.lean |
10 |
12 |
['AntoineChambert-Loir', 'alreadydone', 'github-actions', 'jcommelin', 'leanprover-community-bot-assistant'] |
nobody |
2-15264 2 days ago |
13-19053 13 days ago |
13-19770 13 days |
26667 |
mariainesdff author:mariainesdff |
feat(FieldTheory/SplittingField/IsSplittingField): add IsScalarTower.splits, IsScalarTower.isAlgebraic |
Co-authored-by: @faenuccio
---
- [ ] depends on: #26666
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
29/0 |
Mathlib/Algebra/Polynomial/Lifts.lean,Mathlib/FieldTheory/SplittingField/IsSplittingField.lean |
2 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'tb65536'] |
nobody |
2-12138 2 days ago |
4-51006 4 days ago |
4-51613 4 days |
27244 |
xroblot author:xroblot |
feat(RingTheory/DedekindDomain): lifting an ideal in an extension is injective |
This PR develops some API for [FractionalIdeal.extended](https://leanprover-community.github.io/mathlib4_docs/Mathlib/RingTheory/FractionalIdeal/Extended.html#FractionalIdeal.extended) and in particular for when it is an injective map (for an algebra map). As a consequence, it deduces the fact that lifting an integral ideal in an extension of Dedekind domains is an injective map.
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebra
label:t-algebra$ |
190/5 |
Mathlib/RingTheory/DedekindDomain/Ideal.lean,Mathlib/RingTheory/FractionalIdeal/Extended.lean,Mathlib/RingTheory/Localization/Basic.lean |
3 |
1 |
['github-actions'] |
nobody |
2-1310 2 days ago |
2-2562 2 days ago |
2-2605 2 days |
27230 |
paulorauber author:paulorauber |
feat(Probability): Prove Hoeffding's lemma corollary |
Prove a corollary of Hoeffding's lemma for random variables with non-zero expectation.
This simple corollary was suggested by a reviewer based on a recent contribution (#26744).
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-measure-probability
|
18/9 |
Mathlib/Probability/Moments/SubGaussian.lean |
1 |
1 |
['github-actions'] |
nobody |
2-931 2 days ago |
2-43216 2 days ago |
2-43265 2 days |
23940 |
YaelDillies author:YaelDillies |
feat: polytopes |
From Toric
Co-authored-by: Matthew Johnson
---
[](https://gitpod.io/from-referrer/)
|
toric
t-analysis
|
65/0 |
Mathlib.lean,Mathlib/Geometry/Convex/Polytope.lean,Mathlib/Geometry/Convex/README.md |
3 |
9 |
['Parcly-Taxel', 'YaelDillies', 'eric-wieser', 'github-actions', 'jsm28', 'leanprover-community-bot-assistant'] |
nobody |
1-77034 1 day ago |
38-31579 1 month ago |
99-17301 99 days |
26295 |
DavidJWebb author:DavidJWebb |
feat: filtering lists and bounded quantifiers are primitive recursive |
A few useful lemmas not explicitly in Primrec.lean :
- Filtering for elements from a list that meet a primrec criterion is primrec
- Checking whether a list has some element meeting a primrec criterion is primrec
- Checking whether every element of a list meets a primrec criterion is primrec
- Primitive recursive functions are closed under bounded existential and universal quantifiers
---
[](https://gitpod.io/from-referrer/)
|
t-computability
new-contributor
|
210/0 |
Mathlib.lean,Mathlib/Computability/PrimrecFilter.lean |
2 |
3 |
['DavidJWebb', 'github-actions', 'grunweg'] |
nobody |
1-76022 1 day ago |
25-80880 25 days ago |
25-82570 25 days |
26811 |
loefflerd author:loefflerd |
feat(LinearAlgebra/Projectivization): GL(V) action |
Some API around projective spaces and general linear groups:
- an equiv between V and W gives an equiv between GL(V) and GL(W)
- GL(V) acts on the projectivization of V
- GL 2 K acts on `OnePoint K` (which is the projectivization of `K x K`)
I am adding these because I need them to define cusps in modular form theory, but they are hopefully something of general usefulness beyond that.
---
- [x] depends on: #27104
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebra
label:t-algebra$ |
146/3 |
Mathlib.lean,Mathlib/LinearAlgebra/GeneralLinearGroup.lean,Mathlib/LinearAlgebra/Projectivization/GLAction.lean,Mathlib/Topology/Compactification/OnePoint/ProjectiveLine.lean |
4 |
26 |
['bjoernkjoshanssen', 'eric-wieser', 'github-actions', 'loefflerd', 'mathlib4-dependent-issues-bot'] |
nobody |
1-74740 1 day ago |
4-68864 4 days ago |
13-18757 13 days |
26810 |
oliver-butterley author:oliver-butterley |
feat (Mathlib/Dynamics/BirkhoffSum/Basic): add lemma `birkhoffSum_of_comp_eq` |
If a function `φ` is invariant under a function `f` (i.e., `φ ∘ f = φ`), then the Birkhoff sum of `φ` over `f` for `n` iterations is equal to `n • φ`.
Co-authored-by: Lua Viana Reis
---
- [x] depends on: #26807
[](https://gitpod.io/from-referrer/)
|
t-dynamics
easy
|
9/0 |
Mathlib/Dynamics/BirkhoffSum/Basic.lean |
1 |
4 |
['Ruben-VandeVelde', 'github-actions', 'mathlib4-dependent-issues-bot', 'oliver-butterley'] |
nobody |
1-68363 1 day ago |
1-68363 1 day ago |
12-3331 12 days |
26403 |
riccardobrasca author:riccardobrasca |
feat: add `isPrincipalIdealRing_of_isPrincipal_of_lt_or_isPrincipal_of_mem_primesOver_of_mem_Icc` |
This PR continues the work from #25186.
Original PR: https://github.com/leanprover-community/mathlib4/pull/25186 |
t-number-theory |
48/12 |
Mathlib/NumberTheory/NumberField/ClassNumber.lean |
1 |
3 |
['github-actions', 'riccardobrasca', 'xroblot'] |
nobody |
1-68090 1 day ago |
24-50379 24 days ago |
24-50412 24 days |
27232 |
vihdzp author:vihdzp |
chore: split `Order.Data.Sign` |
We now have a `Defs` file defining `SignType` and basic instances, as well as a `Basic` file proving results about the sign function on a ring.
The files have not been changed beyond updating the module description.
---
A future PR will add `Order.Data.Sign.SuccPred` to this folder.
[](https://gitpod.io/from-referrer/)
|
t-data
tech debt
t-order
|
572/544 |
Mathlib.lean,Mathlib/Data/EReal/Inv.lean,Mathlib/Data/Sign.lean,Mathlib/Data/Sign/Basic.lean,Mathlib/Data/Sign/Defs.lean,Mathlib/LinearAlgebra/AffineSpace/Independent.lean,Mathlib/LinearAlgebra/Matrix/Determinant/TotallyUnimodular.lean,Mathlib/LinearAlgebra/QuadraticForm/Real.lean,Mathlib/Topology/Instances/Sign.lean |
9 |
1 |
['github-actions'] |
nobody |
1-67660 1 day ago |
1-74040 1 day ago |
1-74039 1 day |
26074 |
oliver-butterley author:oliver-butterley |
feat(Mathlib.Dynamics.BirkhoffSum): add 2 lemmas for birkhoffSum/birkhoffAverage concerning ae_eq observables |
If two observables are `ae_eq` then the birkhoffSum/birkhoffAverage of those observables are `ae_eq`.
Motivation:
- Generally it is useful to be able to swap to observables which are `ae_eq`.
- Specifically this is useful to prove Birkhoff's pointwise ergodic theorem by first proving the result for integrable and measurable observables and then using this to deduce the result with just the requirement of integrable.
---
[](https://gitpod.io/from-referrer/)
|
t-dynamics |
44/0 |
Mathlib.lean,Mathlib/Dynamics/BirkhoffSum/QuasiMeasurePreserving.lean |
2 |
10 |
['github-actions', 'oliver-butterley', 'sgouezel'] |
nobody |
1-67567 1 day ago |
1-67585 1 day ago |
31-70435 31 days |
26853 |
oliver-butterley author:oliver-butterley |
feat(Mathlib/MeasureTheory/MeasurableSpace/Invariants): add `comp_eq_of_measurable_invariants` |
Invariance of `g` follows from `Measurable[invariants f] g`.
Co-authored-by: Lua Viana Reis
---
[](https://gitpod.io/from-referrer/)
|
t-measure-probability
easy
|
6/0 |
Mathlib/MeasureTheory/MeasurableSpace/Invariants.lean |
1 |
2 |
['Ruben-VandeVelde', 'github-actions'] |
nobody |
1-66827 1 day ago |
1-66827 1 day ago |
12-19272 12 days |
26840 |
oliver-butterley author:oliver-butterley |
feat(Mathlib/Dynamics/BirkhoffSum/Average): add 3 BirkhoffAverage lemmas |
- `birkhoffAverage_add`
- `birkhoffAverage_neg`
- `birkhoffAverage_sub`
Co-authored-by: Lua Viana Reis
---
[](https://gitpod.io/from-referrer/)
|
t-dynamics |
22/1 |
Mathlib/Dynamics/BirkhoffSum/Average.lean |
1 |
1 |
['github-actions'] |
nobody |
1-66124 1 day ago |
12-74079 12 days ago |
12-74135 12 days |
27123 |
RemyDegenne author:RemyDegenne |
feat: summability results |
- If a real function is summable, then its sum in ENNReal is finite.
- For a real function `f` with `i <= f i` and `c < 0`, `Summable fun i ↦ exp (c * f i)`
---
[](https://gitpod.io/from-referrer/)
|
t-analysis |
15/0 |
Mathlib/Analysis/SpecialFunctions/Exp.lean,Mathlib/Topology/Instances/ENNReal/Lemmas.lean |
2 |
2 |
['RemyDegenne', 'github-actions', 'sgouezel'] |
nobody |
1-61983 1 day ago |
1-62046 1 day ago |
4-13313 4 days |
25874 |
themathqueen author:themathqueen |
feat(LinearAlgebra/Projection): lemmas on projections and invariant submodules |
Proving some lemmas on invariant submodules, such as:
For idempotent `f` and any operator `T`:
- `range f` is invariant under `T` iff `f ∘ T ∘ f = T ∘ f`
- `ker f` is invariant under `T` iff `f ∘ T ∘ f = f ∘ T`
- `f` and `T` commute iff both `range f` and `ker f` are invariant under `T`
Added for both linear maps and continuous linear maps for convenience.
Taken from leanprover-community/mathlib3#18289.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-algebra
label:t-algebra$ |
229/16 |
Mathlib/Algebra/Group/Commute/Units.lean,Mathlib/Algebra/Lie/LieTheorem.lean,Mathlib/Algebra/Module/Submodule/Invariant.lean,Mathlib/Analysis/InnerProductSpace/Projection.lean,Mathlib/LinearAlgebra/Projection.lean,Mathlib/Topology/Algebra/Module/LinearMap.lean |
6 |
45 |
['github-actions', 'j-loreaux', 'leanprover-community-bot-assistant', 'themathqueen'] |
nobody |
1-61977 1 day ago |
1-62668 1 day ago |
26-2941 26 days |
27247 |
RemyDegenne author:RemyDegenne |
feat: measure_inter_eq_of_ae |
For measurable sets `s, t`, if `∀ᵐ a ∂μ, a ∈ t` then `μ (t ∩ s) = μ s`.
From the Brownian motion project.
---
[](https://gitpod.io/from-referrer/)
|
t-measure-probability |
13/0 |
Mathlib/MeasureTheory/Measure/MeasureSpace.lean,Mathlib/MeasureTheory/Measure/Typeclasses/Finite.lean |
2 |
1 |
['github-actions'] |
nobody |
1-60244 1 day ago |
1-60251 1 day ago |
1-60295 1 day |
27246 |
IvanRenison author:IvanRenison |
feat(Analysis/InnerProductSpace/Positive.): add theorems `LinearMap.IsPositive.of_isStarProjection` and `LinearMap.IsIdempotentElem.isPositive_iff_isSelfAdjoint` |
This two theorems where already added for `ContinuousLinearMap`, and in this pull request I'm adding them for `LinearMap`
---
[](https://gitpod.io/from-referrer/)
|
t-analysis |
26/6 |
Mathlib/Analysis/InnerProductSpace/Adjoint.lean,Mathlib/Analysis/InnerProductSpace/Positive.lean |
2 |
6 |
['IvanRenison', 'github-actions', 'themathqueen'] |
nobody |
1-58549 1 day ago |
1-67248 1 day ago |
1-67291 1 day |
27180 |
ADedecker author:ADedecker |
feat: quotient of a monoid with zero by a multiplicative congruence |
---
My motivation is getting a more conceptual construction of [ValuativeRel.ValueGroupWithZero](https://leanprover-community.github.io/mathlib4_docs/Mathlib/RingTheory/Valuation/ValuativeRel.html#ValuativeRel.ValueGroupWithZero), but I think this is of independent interest.
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
141/26 |
Mathlib.lean,Mathlib/Data/Quot.lean,Mathlib/Data/Setoid/Basic.lean,Mathlib/GroupTheory/Congruence/Defs.lean,Mathlib/GroupTheory/Congruence/GroupWithZero.lean |
5 |
22 |
['ADedecker', 'eric-wieser', 'github-actions'] |
nobody |
1-53335 1 day ago |
3-70121 3 days ago |
3-80565 3 days |
27190 |
bwangpj author:bwangpj |
feat(Data/Matrix): matrices with entries in a set |
Define the `Set`/`AddSubmonoid`/`AddSubgroup`/`Subring` of matrices with entries in a `Set`/`AddSubmonoid`/`AddSubgroup`/`Subring`.
---
[](https://gitpod.io/from-referrer/)
|
t-data
new-contributor
|
102/0 |
Mathlib/Data/Matrix/Basic.lean,Mathlib/Data/Matrix/Basis.lean,Mathlib/Data/Matrix/Defs.lean,Mathlib/Data/Matrix/Diagonal.lean |
4 |
20 |
['bwangpj', 'eric-wieser', 'github-actions'] |
nobody |
1-49754 1 day ago |
3-76584 3 days ago |
3-76629 3 days |
27255 |
Louddy author:Louddy |
feat: coeff_mul lemmas |
Add lemmas regarding the interaction of multiplication and the `SkewMonoidAlgebra.coeff`.
Co-authored-by: María Inés de Frutos Fernández <[mariaines.dff@gmail.com](mailto:mariaines.dff@gmail.com)>
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
124/0 |
Mathlib/Algebra/SkewMonoidAlgebra/Basic.lean |
1 |
1 |
['github-actions'] |
nobody |
1-49453 1 day ago |
1-49520 1 day ago |
1-49511 1 day |
27245 |
rirarika author:rirarika |
MvPolynomial.Irreducible |
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-algebra
label:t-algebra$ |
88/0 |
Mathlib.lean,Mathlib/Algebra/MvPolynomial/Irreducible.lean |
2 |
3 |
['alreadydone', 'github-actions', 'mbkybky'] |
nobody |
1-46448 1 day ago |
1-72937 1 day ago |
1-72980 1 day |
26059 |
wwylele author:wwylele |
feat(GroupTheory/Divisible): Add rational SMul and Module |
This is part of https://github.com/leanprover-community/mathlib4/pull/25140. A torsion-free ℕ-divisible commutative group is a ℚ-module.
----
This PR continues the work from #25190.
Original PR: https://github.com/leanprover-community/mathlib4/pull/25190 |
t-algebra label:t-algebra$ |
156/0 |
Mathlib/Data/NNRat/Lemmas.lean,Mathlib/Data/Rat/Lemmas.lean,Mathlib/GroupTheory/Divisible.lean |
3 |
5 |
['eric-wieser', 'github-actions', 'wwylele'] |
nobody |
1-45683 1 day ago |
32-12941 1 month ago |
32-12961 32 days |
27257 |
JovanGerb author:JovanGerb |
feat(LinearAlgebra/AffineSpace/Ordered): add `lineMap_le_lineMap_iff_of_lt'` |
I only need `lineMap_le_lineMap_iff_of_lt'`. The other lemmas are added for completeness.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
16/0 |
Mathlib/LinearAlgebra/AffineSpace/Ordered.lean |
1 |
1 |
['github-actions'] |
nobody |
1-41603 1 day ago |
1-41648 1 day ago |
1-41780 1 day |
26975 |
Whysoserioushah author:Whysoserioushah |
feat: a norm_num extension for complex numbers |
co-authored-by : @thefundamentaltheor3m, @hrmacbeth
---
[](https://gitpod.io/from-referrer/)
|
t-meta |
337/0 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/NormNum/NormNumI.lean,MathlibTest/norm_numI.lean |
4 |
35 |
['Whysoserioushah', 'eric-wieser', 'github-actions', 'hrmacbeth'] |
nobody |
1-32338 1 day ago |
2-35816 2 days ago |
2-40133 2 days |
26912 |
pechersky author:pechersky |
chore(Algebra/Ring/Subring): simp tag `Subring.smul_def` |
Ported from #25308
---
[](https://gitpod.io/from-referrer/)
I found this being not-simp frustrating when talking about submodules over a valuation subring. |
t-algebra label:t-algebra$ |
35/39 |
Mathlib/Algebra/Algebra/Subalgebra/Basic.lean,Mathlib/Algebra/Field/Subfield/Basic.lean,Mathlib/Algebra/Group/Subgroup/Actions.lean,Mathlib/Algebra/Group/Submonoid/MulAction.lean,Mathlib/Algebra/Module/LocalizedModule/Basic.lean,Mathlib/Algebra/Module/LocalizedModule/IsLocalization.lean,Mathlib/Algebra/Module/LocalizedModule/Submodule.lean,Mathlib/Algebra/Ring/Periodic.lean,Mathlib/Algebra/Ring/Subring/Basic.lean,Mathlib/Algebra/Ring/Subsemiring/Basic.lean,Mathlib/Analysis/CStarAlgebra/Basic.lean,Mathlib/FieldTheory/KummerExtension.lean,Mathlib/GroupTheory/GroupAction/Defs.lean,Mathlib/GroupTheory/GroupAction/MultiplePrimitivity.lean,Mathlib/GroupTheory/GroupAction/MultipleTransitivity.lean,Mathlib/GroupTheory/GroupAction/SubMulAction/OfFixingSubgroup.lean,Mathlib/GroupTheory/GroupAction/SubMulAction/OfStabilizer.lean,Mathlib/LinearAlgebra/RootSystem/Irreducible.lean,Mathlib/LinearAlgebra/RootSystem/RootPositive.lean,Mathlib/LinearAlgebra/RootSystem/WeylGroup.lean,Mathlib/RingTheory/Localization/InvSubmonoid.lean,Mathlib/RingTheory/OreLocalization/Basic.lean |
22 |
8 |
['github-actions', 'j-loreaux', 'linesthatinterlace', 'pechersky'] |
nobody |
1-31177 1 day ago |
5-79800 5 days ago |
9-17102 9 days |
27055 |
wwylele author:wwylele |
feat(RingTheory): add HahnSeries.truncate |
---
This is for the proof of Hahn embedding theorem #27043, but it feels niche to have it in HahnSeries file, so I am not sure... if this doesn't feel right, I could make them private to the proof.
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
31/0 |
Mathlib/RingTheory/HahnSeries/Addition.lean,Mathlib/RingTheory/HahnSeries/Basic.lean |
2 |
2 |
['ScottCarnahan', 'github-actions'] |
nobody |
1-29098 1 day ago |
7-5237 7 days ago |
7-5285 7 days |
27248 |
kckennylau author:kckennylau |
chore: remove `suppress_compilation` from Mathlib.Algebra.Category.Ring.Constructions |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
easy
label:t-algebra$ |
2/4 |
Mathlib/Algebra/Category/Ring/Constructions.lean |
1 |
4 |
['github-actions', 'grunweg', 'leanprover-bot'] |
nobody |
1-28301 1 day ago |
1-60185 1 day ago |
1-60233 1 day |
27249 |
pechersky author:pechersky |
feat(Topology/Completion): coe_inj and simp lemmas for coe zero and one |
---
[](https://gitpod.io/from-referrer/)
|
t-analysis
t-topology
easy
|
11/0 |
Mathlib/Topology/Algebra/GroupCompletion.lean,Mathlib/Topology/Algebra/UniformRing.lean,Mathlib/Topology/UniformSpace/Completion.lean |
3 |
1 |
['github-actions'] |
nobody |
1-25483 1 day ago |
1-59075 1 day ago |
1-59117 1 day |
27261 |
Sebi-Kumar author:Sebi-Kumar |
feat(Topology): add definition for subpaths |
Define subpaths as restrictions of paths to subintervals, reparameterized to have domain
`[0, 1]` and possibly with a reverse of direction. Prove their basic properties.
This serves as an alternative to `Path.truncate` which is useful for the explicit construction of certain homotopies, in particular regarding the concatenation of subpaths.
---
To provide additional context, this is my first time contributing to Mathlib,
and I am doing so as a part of the Fields Undergraduate Summer Research Program
hosted at Western University.
My intention for this file is for it to be used when proving that the fundamental group of the sphere is trivial (following the proof from Hatcher's "Algebraic Topology").
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-topology
|
148/0 |
Mathlib.lean,Mathlib/Topology/Subpath.lean |
2 |
1 |
['github-actions'] |
nobody |
1-25471 1 day ago |
1-36102 1 day ago |
1-36149 1 day |
27264 |
pechersky author:pechersky |
feat(Topology/ValuedField): range of valuation on competion is the same as base field |
and other helper API to prepare for ValuativeTopology
---
[](https://gitpod.io/from-referrer/)
|
t-topology |
60/0 |
Mathlib/Topology/Algebra/Valued/ValuedField.lean |
1 |
1 |
['github-actions'] |
nobody |
1-24320 1 day ago |
1-24330 1 day ago |
1-24374 1 day |
27265 |
pechersky author:pechersky |
feat(Topology/Valued): discrete topology on a valued field when trivial valuation |
or when there is a nonzero term in the valuation codomain that is smaller than all nonzero valuations
---
[](https://gitpod.io/from-referrer/)
|
t-topology |
33/0 |
Mathlib/Topology/Algebra/Valued/ValuationTopology.lean |
1 |
1 |
['github-actions'] |
nobody |
1-24316 1 day ago |
1-24320 1 day ago |
1-24363 1 day |
25833 |
loefflerd author:loefflerd |
feat(Counterexamples): topologists' sine curve |
Define the "topologists' sine curve" in R^2, and show that its closure is connected but not path-connected.
This formalization is part of the bachelor thesis of Daniele Bolla at UniDistance Switzerland.
Co-authored-by: Daniele Bolla [daniele.bolla@stu.fernuni.ch](mailto:daniele.bolla@stu.fernuni.ch)
---
[](https://gitpod.io/from-referrer/)
|
migrated-from-branch
t-topology
|
219/1 |
Counterexamples.lean,Counterexamples/TopologistsSineCurve.lean,Mathlib/Topology/Connected/PathConnected.lean |
3 |
13 |
['Ruben-VandeVelde', 'github-actions', 'loefflerd', 'sgouezel'] |
nobody |
1-22751 1 day ago |
1-22884 1 day ago |
36-57042 36 days |
27172 |
pechersky author:pechersky |
feat(Order/DenselyOrderedLocallyFinite): linear locally finite dense orders are trivial |
---
[](https://gitpod.io/from-referrer/)
- [x] depends on: #27170
- [x] depends on: #27171 |
t-order |
169/2 |
Mathlib.lean,Mathlib/Data/Set/Subsingleton.lean,Mathlib/GroupTheory/ArchimedeanDensely.lean,Mathlib/Order/Basic.lean,Mathlib/Order/DenselyOrderedLocallyFinite.lean |
5 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
1-20298 1 day ago |
1-22364 1 day ago |
1-22645 1 day |
26704 |
euprunin author:euprunin |
chore: golf Algebra/ using `aesop` |
|
t-algebra label:t-algebra$ |
10/36 |
Mathlib/Algebra/Colimit/Ring.lean,Mathlib/Algebra/Group/Submonoid/BigOperators.lean,Mathlib/Algebra/GroupWithZero/Regular.lean,Mathlib/Algebra/Homology/Embedding/Basic.lean,Mathlib/Algebra/Homology/Embedding/Connect.lean,Mathlib/Algebra/Lie/Ideal.lean,Mathlib/Algebra/MvPolynomial/Equiv.lean,Mathlib/Algebra/Polynomial/Reverse.lean |
8 |
25 |
['euprunin', 'github-actions', 'grunweg', 'leanprover-bot', 'leanprover-community-bot-assistant', 'leanprover-community-mathlib4-bot'] |
nobody |
1-19781 1 day ago |
1-19781 1 day ago |
11-6337 11 days |
27057 |
AntoineChambert-Loir author:AntoineChambert-Loir |
feat(GroupTheory/SpecificGroups/Alternating/KleinFour): the Klein Four subgroup of alternatingGroup on 4 letters |
Let `α` be a finite type.
* `alternatingGroup.center_eq_bot`: when `4 ≤ Nat.card α`, then center of `alternatingGroup α` is trivial.
We now assume that `Nat.card α = 4`.
* `alternatingGroup.kleinFour` : the subgroup of `alternatingGroup α` generated by permutations of cycle type (2, 2).
* `alternatingGroup.kleinFour_isKleinFour`:`alternatingGroup.kleinFour α` satisfies `IsKleinFour`.
(When `4 < Nat.card α`, it is equal to `⊤`, when `Nat.card α < 4`, it is trivial.)
* `alternatingGroup.two_sylow_eq_kleinFour_of_four`:
All `2`-sylow subgroups of `alternatingGroup α` are equal to `kleinFour α`.
* `alternatingGroup.characteristic_kleinFour`: the subgroup `alternatingGroup.kleinFour α` is characteristic.
* `alternatingGroup.normal_kleinFour`: the subgroup `alternatingGroup.kleinFour α` is normal.
* `alternatingGroup.kleinFour_eq_commutator`:
the subgroup `alternatingGroup.kleinFour α` is the commutator subgroup of `alternatingGroup α`.
(When `4 < Nat.card α`, the commutator subgroup of `alternatingGroup α` is equal to `⊤`; when `Nat.card α < 3`, it is trivial.)
## Remark on implementation
We start from `kleinFour α` as given by its definition.
We first prove that it is equal to any 2-sylow subgroup: the elements of such a sylow subgroup `S` have order a power of 2, and this implies that their cycle type is () or (2,2).
Since there are exactly 4 elements of that cycle type, we conclude that `kleinFour α = S`.
Since all 2-sylow subgroups are conjugate, we conclude that there is only one 2-sylow subgroup and that it is normal, and then characteristic.
## TODO :
Prove `alternatingGroup.kleinFour α = commutator (alternatingGroup α)` without any assumption on `Nat.card α`.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
322/1 |
Mathlib.lean,Mathlib/GroupTheory/Abelianization.lean,Mathlib/GroupTheory/SpecificGroups/Alternating.lean,Mathlib/GroupTheory/SpecificGroups/Alternating/KleinFour.lean,Mathlib/GroupTheory/Sylow.lean |
5 |
15 |
['AntoineChambert-Loir', 'github-actions', 'tb65536'] |
nobody |
1-16828 1 day ago |
6-82222 6 days ago |
6-82265 6 days |
26243 |
DavidLedvinka author:DavidLedvinka |
feat(Topology): Add PairReduction.lean |
Add file PairReduction.lean which proves the theorem `pair_reduction` which is needed for the proof of the general Kolmogorov-Chentsov theorem in the Brownian Motion project.
Co-authored-by: @RemyDegenne
- [ ] depends on: #27239 |
t-topology |
400/0 |
Mathlib.lean,Mathlib/Topology/EMetricSpace/PairReduction.lean |
2 |
65 |
['DavidLedvinka', 'EtienneC30', 'RemyDegenne', 'github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
1-16012 1 day ago |
1-51060 1 day ago |
28-35944 28 days |
26114 |
wwylele author:wwylele |
feat(Data/Real): add embedding of archimedean groups into Real |
This is part of https://github.com/leanprover-community/mathlib4/pull/25140, and is the special case of Hahn embedding theorem applied to archimedean group.
----
This PR continues the work from #25157.
Original PR: https://github.com/leanprover-community/mathlib4/pull/25157 |
t-data |
231/0 |
Mathlib.lean,Mathlib/Data/Rat/Lemmas.lean,Mathlib/Data/Real/Embedding.lean |
3 |
21 |
['ScottCarnahan', 'github-actions', 'wwylele'] |
nobody |
1-15532 1 day ago |
31-38213 1 month ago |
31-38259 31 days |
27241 |
alreadydone author:alreadydone |
feat(MonoidAlgebra): generalize IsDomain instance |
The instance works over a semiring with cancellative addition. It's then used to generalize the IsDomain instances on Polynomial and MvPolynomial.
---
- [x] depends on: #27263
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
78/69 |
Mathlib/Algebra/MonoidAlgebra/NoZeroDivisors.lean,Mathlib/Algebra/MvPolynomial/Basic.lean,Mathlib/Algebra/MvPolynomial/Funext.lean,Mathlib/Algebra/Polynomial/Basic.lean,Mathlib/Algebra/Polynomial/Degree/Domain.lean,Mathlib/FieldTheory/RatFunc/Defs.lean,Mathlib/LinearAlgebra/Matrix/Adjugate.lean,Mathlib/LinearAlgebra/Vandermonde.lean,Mathlib/RingTheory/Polynomial/Basic.lean |
9 |
24 |
['YaelDillies', 'alreadydone', 'eric-wieser', 'github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
1-12934 1 day ago |
1-12936 1 day ago |
1-81749 1 day |
27142 |
YaelDillies author:YaelDillies |
feat(LinearAlgebra/TensorProduct): `map f₂ g₂ (map f₁ g₁ x) = map (f₂ ∘ₗ f₁) (g₂ ∘ₗ g₁) x` |
From Toric
---
[](https://gitpod.io/from-referrer/)
|
toric
t-algebra
label:t-algebra$ |
14/5 |
Mathlib/LinearAlgebra/TensorProduct/Basic.lean |
1 |
4 |
['YaelDillies', 'eric-wieser', 'github-actions'] |
nobody |
1-9181 1 day ago |
5-43057 5 days ago |
5-43047 5 days |
26484 |
peabrainiac author:peabrainiac |
feat(Geometry/Diffeology): basics of diffeological spaces |
Introduces diffeological spaces, smooth maps between them, the D-topology and the standard diffeology on finite-dimensional normed spaces.
---
This PR continues the work from #21969. |
t-differential-geometry |
471/0 |
Mathlib.lean,Mathlib/Geometry/Diffeology/Basic.lean,docs/references.bib |
3 |
9 |
['JovanGerb', 'github-actions', 'lecopivo', 'peabrainiac'] |
nobody |
1-7220 1 day ago |
22-4538 22 days ago |
22-9290 22 days |
25920 |
BoltonBailey author:BoltonBailey |
feat(Data/Finsupp/Basic): `Finsupp.optionElim'` |
Similar to how Finsupp.cons constructs a map Fin (n + 1) →₀ M from a map Fin n →₀ M,
we define Finsupp.optionElim' to construct a map Option α →₀ M from a map α →₀ M, given an additional value for none. We base this on the new optionEquiv definition. As a function, it behaves as Option.elim', hence the name.
We prove a variety of API lemmas, based on those for Finsupp.cons, to bring the definitions more in line with the contents of Data/Finsupp/Fin.
We also refactor to a new file to help avoid a too-long file and make this more analogous to Finsupp.cons
Original PR: https://github.com/leanprover-community/mathlib4/pull/13861
- [x] depends on: #26309 |
migrated-from-branch
t-data
|
124/25 |
Mathlib/Algebra/Category/MonCat/Adjunctions.lean,Mathlib/Data/Finsupp/Option.lean |
2 |
13 |
['BoltonBailey', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
1-4685 1 day ago |
1-4705 1 day ago |
23-11688 23 days |
27105 |
xroblot author:xroblot |
feat(Ring/DedekindDomain): formula for the splitting of prime ideals in an extension |
This PR just puts together all the results that were already there to deduce:
```lean
map (algebraMap S R) p = ∏ P ∈ p.primesOver R, P ^ p.ramificationIdx (algebraMap S R) P
```
for `p` a maximal ideal of a ring `S` and `R` an extension of `S` that is a Dedekind ring.
Note. There is a significant import increase in the file `RingTheory.DedekindDomain.Factorization`. However, this file is almost a leaf file so this increase only affects a limited number of files. If the increase is too big, a new file, say `RingTheory.DedekindDomain.PrimeSplitting`, can be added instead.
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebra
label:t-algebra$ |
89/3 |
Mathlib/RingTheory/DedekindDomain/Factorization.lean,Mathlib/RingTheory/DedekindDomain/Ideal.lean,Mathlib/RingTheory/Ideal/Operations.lean,Mathlib/RingTheory/Ideal/Over.lean |
4 |
1 |
['github-actions'] |
nobody |
1-2260 1 day ago |
6-10617 6 days ago |
6-10661 6 days |
27266 |
euprunin author:euprunin |
chore: use `simp` or `simp_all` instead of `aesop` in Algebra/ |
Motivation: reducing overhead and clarifying intent. |
t-algebra label:t-algebra$ |
17/17 |
Mathlib/Algebra/BigOperators/Finprod.lean,Mathlib/Algebra/BigOperators/Group/List/Basic.lean,Mathlib/Algebra/DirectSum/Internal.lean,Mathlib/Algebra/Group/Pointwise/Finset/Basic.lean,Mathlib/Algebra/GroupWithZero/Associated.lean,Mathlib/Algebra/Lie/TraceForm.lean,Mathlib/Algebra/Module/CharacterModule.lean,Mathlib/Algebra/Module/Submodule/Range.lean,Mathlib/Algebra/MvPolynomial/Basic.lean,Mathlib/Algebra/Order/Antidiag/Nat.lean,Mathlib/Algebra/Order/Antidiag/Pi.lean,Mathlib/Algebra/Order/Ring/Star.lean,Mathlib/Algebra/Polynomial/Degree/Definitions.lean,Mathlib/Algebra/Polynomial/Degree/Lemmas.lean,Mathlib/Algebra/Polynomial/Degree/Monomial.lean,Mathlib/Algebra/Polynomial/SpecificDegree.lean |
16 |
1 |
['github-actions'] |
nobody |
0-85457 23 hours ago |
1-22905 1 day ago |
1-22949 1 day |
26793 |
FlAmmmmING author:FlAmmmmING |
feat(Algebra/Group /ForwardDiff.lean): add five theorems for forward difference |
---
[](https://gitpod.io/from-referrer/)
|
large-import
new-contributor
t-algebra
label:t-algebra$ |
212/3 |
Mathlib/Algebra/Group/ForwardDiff.lean |
1 |
35 |
['AntoineChambert-Loir', 'DAE123456', 'FlAmmmmING', 'Ruben-VandeVelde', 'github-actions', 'kckennylau', 'madvorak'] |
nobody |
0-76452 21 hours ago |
2-3006 2 days ago |
14-41893 14 days |
27253 |
Louddy author:Louddy |
feat: SkewMonoidAlgebra/Support |
Add lemmas regarding the support of a skew monoid algebra.
It is currently missing a few lemmas compared to `MonoidAlgebra.support`. (See TODO.)
These will be added as more results are available on `SkewMonoidAlgebra`.
Co-authored-by: María Inés de Frutos Fernández <[mariaines.dff@gmail.com](mailto:mariaines.dff@gmail.com)>
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
100/0 |
Mathlib.lean,Mathlib/Algebra/SkewMonoidAlgebra/Support.lean |
2 |
1 |
['github-actions'] |
nobody |
0-75241 20 hours ago |
1-50957 1 day ago |
1-50969 1 day |
27283 |
Louddy author:Louddy |
feat: maps on/to SkewMonoidAlgebra |
Add the definition of many maps regarding skew monoid algebras and lemmas associated to them. These all have their analogues for `MonoidAlgebra`.
Co-authored-by: María Inés de Frutos Fernández <[mariaines.dff@gmail.com](mailto:mariaines.dff@gmail.com)>
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebra
label:t-algebra$ |
237/0 |
Mathlib/Algebra/SkewMonoidAlgebra/Basic.lean |
1 |
1 |
['github-actions'] |
nobody |
0-75023 20 hours ago |
0-75029 20 hours ago |
0-75078 20 hours |
27284 |
FernandoChu author:FernandoChu |
Chore(CategoryTheory/MorphismProperty/MonoFactorization): Factor out mono factorizations |
Factored out `MonoFactorisations` from the `Images` file; also rename it to `MonoFactori*z*ations` so it's inline with the rest of Mathlib. I'm also sneaking in some very basic extremal epis results if you don't mind, these were meant to be used to prove
```lean
instance (priority := 100) hasStrongEpiImages_of_hasPullbacks_of_hasEqualizers [HasPullbacks C]
[HasEqualizers C] : HasStrongEpiImages C
```
Which I noticed too late already had a proof; I think the proof has been improved anyways, it's just `infer_instance` now. |
new-contributor
t-category-theory
|
419/259 |
Mathlib.lean,Mathlib/Algebra/Category/Grp/Images.lean,Mathlib/Algebra/Category/ModuleCat/Images.lean,Mathlib/AlgebraicTopology/SimplexCategory/Basic.lean,Mathlib/CategoryTheory/Abelian/Basic.lean,Mathlib/CategoryTheory/Category/Factorisation.lean,Mathlib/CategoryTheory/ConcreteCategory/EpiMono.lean,Mathlib/CategoryTheory/Limits/Preserves/Shapes/Images.lean,Mathlib/CategoryTheory/Limits/Shapes/ExtremalEpi.lean,Mathlib/CategoryTheory/Limits/Shapes/Images.lean,Mathlib/CategoryTheory/Limits/Shapes/Kernels.lean,Mathlib/CategoryTheory/Limits/Shapes/StrongEpi.lean,Mathlib/CategoryTheory/Limits/Shapes/ZeroMorphisms.lean,Mathlib/CategoryTheory/Limits/Types/Images.lean,Mathlib/CategoryTheory/MorphismProperty/MonoFactorization.lean,Mathlib/CategoryTheory/Sites/Subsheaf.lean,Mathlib/Order/Category/NonemptyFinLinOrd.lean,scripts/nolints_prime_decls.txt |
18 |
1 |
['github-actions'] |
nobody |
0-69655 19 hours ago |
0-72213 20 hours ago |
0-72263 20 hours |
27260 |
JovanGerb author:JovanGerb |
feat(Geometry/Euclidean/SignedDist): `signedDist` between two points |
original PR: #24245
This PR defines `signedDist`, the signed distance between two points.
TODO: It redefines `signedInfDist` so that it uses `signedDist`.
The motivation is to use this in IMO2020Q6. Additionally this definition will be useful for properly reasoning about the power of a point
[#mathlib4 > Signed distance between points](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Signed.20distance.20between.20points)
some comments:
* should `signedDistLinear` be `private`?
* I'm not too happy about the hypothesis in `signedDist_congr (h : ∃ r > (0 : ℝ), r • v = w)`. This relationship between `v` and `w` is a symmetric one that should have some API around it, similar to `SameRay`. It could also be spelled as `(ℝ≥0 ∙ v) = ℝ≥0 ∙ w`
---
- [x] depends on: #27259
- [ ] depends on : #27285
[](https://gitpod.io/from-referrer/)
|
|
207/30 |
Mathlib/Analysis/InnerProductSpace/Basic.lean,Mathlib/Analysis/Normed/Lp/ProdLp.lean,Mathlib/Geometry/Euclidean/SignedDist.lean,Mathlib/Topology/MetricSpace/Pseudo/Defs.lean |
4 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
0-64758 17 hours ago |
0-67309 18 hours ago |
0-73885 20 hours |
25500 |
eric-wieser author:eric-wieser |
feat: delaborators for metadata |
Being able to see these is very important when debugging tactic failures. Probably these could be upstreamed, but I don't think that's a reason not to merge them here first.
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-meta
|
75/3 |
Mathlib/Util/Delaborators.lean,Mathlib/Util/PPOptions.lean,MathlibTest/delaborators.lean |
3 |
11 |
['JovanGerb', 'Rob23oba', 'eric-wieser', 'github-actions'] |
nobody |
0-57713 16 hours ago |
44-26254 1 month ago |
44-26312 44 days |
27289 |
kckennylau author:kckennylau |
feat(FieldTheory): lemmas about trace and norm in finite fields |
---
Zulip: [#new members > How to formalize a finite field exercise?](https://leanprover.zulipchat.com/#narrow/channel/113489-new-members/topic/How.20to.20formalize.20a.20finite.20field.20exercise.3F/with/529553211)
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
41/4 |
Mathlib/FieldTheory/Finite/Basic.lean,Mathlib/FieldTheory/Finite/Trace.lean |
2 |
1 |
['github-actions'] |
nobody |
0-56093 15 hours ago |
0-56448 15 hours ago |
0-56491 15 hours |
27089 |
themathqueen author:themathqueen |
refactor(Analysis/InnerProductSpace/Positive): changing positivity on linear maps to use `IsSymmetric` instead of finite-dimensional and `IsSelfAdjoint` |
With this definition, the partial order would be defined on linear maps without needing finite-dimensionality.
Also, when continuous linear maps are positive, then so are their coercions into linear maps, without needing finite-dimensionality. Moving the definition of positivity for linear maps before the one for continuous linear maps allows us to use results already done in linear maps to golf proofs for continuous linear maps. There's no need to have duplicate proofs.
---
[](https://gitpod.io/from-referrer/)
|
t-analysis |
173/190 |
Mathlib/Analysis/InnerProductSpace/Positive.lean,Mathlib/Analysis/InnerProductSpace/Symmetric.lean |
2 |
7 |
['IvanRenison', 'github-actions', 'leanprover-community-bot-assistant'] |
nobody |
0-55179 15 hours ago |
0-55202 15 hours ago |
6-8601 6 days |
27272 |
eric-wieser author:eric-wieser |
chore: generalize `sumAddHom` to `sumZeroHom` |
This hopefully will make this usable on quadratic maps, which preserve zero but not addition.
For now this does not change the simp-normal form of `sumAddHom`
---
[](https://gitpod.io/from-referrer/)
|
t-data
t-algebra
label:t-algebra$ |
45/24 |
Mathlib/Data/DFinsupp/BigOperators.lean |
1 |
1 |
['github-actions'] |
nobody |
0-53672 14 hours ago |
1-14411 1 day ago |
1-14452 1 day |
27285 |
JovanGerb author:JovanGerb |
feat(MetricSpace): tag `dist_nonneg` with `@[simp]` |
`dist_pos` is already a simp lemma, so `dist_nonneg` should be too.
---
[](https://gitpod.io/from-referrer/)
|
easy |
7/7 |
Mathlib/Analysis/Normed/Lp/ProdLp.lean,Mathlib/Topology/ContinuousMap/Bounded/Basic.lean,Mathlib/Topology/MetricSpace/HausdorffDistance.lean,Mathlib/Topology/MetricSpace/PiNat.lean,Mathlib/Topology/MetricSpace/Pseudo/Constructions.lean,Mathlib/Topology/MetricSpace/Pseudo/Defs.lean |
6 |
1 |
['github-actions'] |
nobody |
0-53599 14 hours ago |
0-53599 14 hours ago |
0-66489 18 hours |
26371 |
Timeroot author:Timeroot |
feat(NumberTheory): Niven's theorem |
This file proves Niven's theorem, that the only rational cosines of angles that are rational multiples of pi, are [-1, -1/2, 0, 1/2, 1]. This is one of the theorems missing from 1000.yaml.
---
[](https://gitpod.io/from-referrer/)
|
t-number-theory |
119/0 |
Mathlib.lean,Mathlib/NumberTheory/Niven.lean,docs/1000.yaml |
3 |
9 |
['Timeroot', 'github-actions', 'grunweg', 'plp127'] |
nobody |
0-53328 14 hours ago |
25-32714 25 days ago |
25-32761 25 days |
27288 |
themathqueen author:themathqueen |
feat(LinearAlgebra/TensorProduct/Basic): add semi-linear versions for `map` and `lift` |
This is for defining the inner product on tensor products: #27228. Also for defining star on tensor products: #27290.
Trying to semi-linearize `LinearAlgebra/TensorProduct/Basic` like the WIP #24208 seems like a big load of work, so, for now, I added `TensorProduct.liftₛₗ` and `TensorProduct.mapₛₗ` for the semi-linear versions, as we need them now.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
41/10 |
Mathlib/LinearAlgebra/TensorProduct/Basic.lean |
1 |
2 |
['eric-wieser', 'github-actions'] |
nobody |
0-52923 14 hours ago |
0-56552 15 hours ago |
0-56603 15 hours |
25347 |
sgouezel author:sgouezel |
feat: define Riemannian manifolds |
We introduce typeclasses to deal with Riemannian manifolds:
* In a fiber bundle whose fibers are already endowed with an inner product space structure, `[IsContinuousRiemannianBundle F E]` registers the fact the inner product depends continuously on the base point. This is a Prop-valued class, on top of existing data `[∀ x, NormedAddCommGroup (E x)]` `[∀ x, InnerProductSpace ℝ (E x)]`.
* We also register `[IsContMDiffRiemannianBundle n IB F E]` similarly.
* There is an issue when the fibers already have a topological structure (for instance the tangent spaces), because adding an assumption `[∀ x, NormedAddCommGroup (TangentSpace I x)]` would create a diamond. Instead, we introduce another typeclass `[RiemannianBundle E]` containing the data of an inner product space on the fibers, compatible with the preexisting topology. From this class, we register instances of inner product space structures on the fibers, whose topology is defeq to the original one.
* We make sure that registering concrete instances of `[RiemannianBundle E]` registers automatically `[IsContinuousRiemannianBundle F E]` and/or `[IsContMDiffRiemannianBundle n IB F E]` in terms of the regularity of the metric.
* Under the assumptions `[RiemannianBundle (fun (b : M) -> TangentSpace I b)]` and `[EMetricSpace M]`, we register a Prop-valued typeclass `[IsRiemannianManifold I M]` registering the fact that the edist coincides with the infimum of the lengths of paths, measured using the normed space structure in the tangent spaces.
With this design, one can develop the general theory of Riemannian bundles and Riemannian manifolds, and also define concrete instances. When working with a generic Riemannian manifold, the typeclasses will include (in addition to the usual one for manifolds, replacing the topological space one with an emetric space one) the assumptions
`[RiemannianBundle (fun (b : M) -> TangentSpace I b)]` `[IsContinuousRiemannianBundle E (fun (b : M) -> TangentSpace I b)]` `[IsContMDiffRiemannianBundle n I E (fun (b : M) -> TangentSpace I b)]`.
---
- [x] depends on: #25383
- [x] depends on: #25768
- [x] depends on: #25771
- [x] depends on: #25824
- [x] depends on: #25865
- [x] depends on: #26066
- [x] depends on: #26068
- [x] depends on: #26069
- [x] depends on: #26112
- [x] depends on: #26113
- [x] depends on: #26121
- [x] depends on: #26198
- [x] depends on: #26197
- [x] depends on: #26356
- [x] depends on: #26362
- [x] depends on: #26361
- [x] depends on: #26355
- [x] depends on: #26411
- [x] depends on: #26500
- [x] depends on: #26501
- [x] depends on: #26502
- [x] depends on: #26503
- [x] depends on: #26504
- [x] depends on: #26505
- [x] depends on: #26506
- [x] depends on: #26778
[](https://gitpod.io/from-referrer/)
|
t-differential-geometry |
587/4 |
Mathlib.lean,Mathlib/Geometry/Manifold/ContMDiff/NormedSpace.lean,Mathlib/Geometry/Manifold/Riemannian/Basic.lean |
3 |
n/a |
['PatrickMassot', 'github-actions', 'grunweg', 'leanprover-bot', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'sgouezel'] |
nobody |
0-51208 14 hours ago |
unknown |
unknown |
27277 |
artie2000 author:artie2000 |
feat(Logic/Equiv): `Equiv` on `Subtype` implies equivalence of existence statements |
* Add lemmas stating that an `Equiv` between `Subtypes` implies the equivalence of the corresponding `Exists` and `ExistsUnique` propositions.
---
[](https://gitpod.io/from-referrer/)
|
t-data |
9/0 |
Mathlib/Logic/Equiv/Defs.lean |
1 |
4 |
['YaelDillies', 'artie2000', 'github-actions'] |
nobody |
0-48547 13 hours ago |
1-3845 1 day ago |
1-6064 1 day |
27254 |
yuanyi-350 author:yuanyi-350 |
2025 imo problem3 |
---
[](https://gitpod.io/from-referrer/)
|
IMO |
370/3 |
Archive.lean,Archive/Imo/Imo2025Q3.lean,Mathlib/Algebra/GeomSum.lean,Mathlib/Algebra/Ring/Int/Parity.lean,Mathlib/Algebra/Ring/Parity.lean,Mathlib/FieldTheory/Finite/Basic.lean,Mathlib/NumberTheory/Multiplicity.lean |
7 |
1 |
['github-actions'] |
nobody |
0-44204 12 hours ago |
0-44260 12 hours ago |
0-44266 12 hours |
26646 |
eric-wieser author:eric-wieser |
feat(TensorProduct): add a Repr |
Now that tensor products are computable again, this makes them `#eval`able.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-meta
label:t-algebra$ |
8/0 |
Mathlib/LinearAlgebra/TensorProduct/Basic.lean |
1 |
6 |
['JovanGerb', 'eric-wieser', 'github-actions'] |
nobody |
0-41602 11 hours ago |
17-9697 17 days ago |
17-9749 17 days |
27279 |
artie2000 author:artie2000 |
feat(FieldTheory): isomorphism with quotient of polynomial ring by minimal polynomial of primitive element |
Define the `F`-isomorphism between a field extension `E/F` and the quotient of `F[X]` by the ideal generated by the minimal polynomial of a primitive element in `E`
---
This PR is technically independent of #27278, but depends on that PR for the isomorphism defined here to have good `simp` properties.
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
32/4 |
Mathlib/FieldTheory/IntermediateField/Adjoin/Algebra.lean,Mathlib/FieldTheory/PrimitiveElement.lean |
2 |
5 |
['YaelDillies', 'artie2000', 'github-actions'] |
nobody |
0-37828 10 hours ago |
0-83049 23 hours ago |
0-83046 23 hours |
27236 |
alreadydone author:alreadydone |
feat(RingTheory): principal ideal product rings |
---
[](https://gitpod.io/from-referrer/)
|
maintainer-merge
t-algebra
easy
label:t-algebra$ |
18/2 |
Mathlib/RingTheory/Ideal/Prod.lean,Mathlib/RingTheory/PrincipalIdealDomain.lean |
2 |
3 |
['YaelDillies', 'github-actions', 'xhalo32'] |
nobody |
0-37094 10 hours ago |
0-37094 10 hours ago |
2-33854 2 days |
27101 |
Paul-Lez author:Paul-Lez |
feat(Tactic/Simproc/Divisors): add `simproc`s to compute the divisors of a natural number. |
This PR continues the work from #23026.
Original PR: https://github.com/leanprover-community/mathlib4/pull/23026 |
t-meta |
76/0 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Simproc/Divisors.lean,MathlibTest/Simproc/Divisors.lean |
4 |
26 |
['Paul-Lez', 'eric-wieser', 'github-actions', 'mathlib-bors', 'plp127'] |
nobody |
0-36655 10 hours ago |
5-17523 5 days ago |
6-17246 6 days |
25292 |
YaelDillies author:YaelDillies |
feat: the `ConvexCone` generated by a set |
Define `ConvexCone.copy` and `ConvexCone.hull` and use them to golf the `CompleteLattice` instance.
From Toric
---
- [x] depends on: #25291
[](https://gitpod.io/from-referrer/)
|
t-convex-geometry
toric
|
90/35 |
Mathlib/Analysis/Convex/Cone/Basic.lean,Mathlib/Geometry/Convex/Cone/Basic.lean |
2 |
4 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
0-36177 10 hours ago |
0-36211 10 hours ago |
30-60395 30 days |
27098 |
Paul-Lez author:Paul-Lez |
feat(Algebra/Category/ModuleCat/Sheaf/VectorBundle): define vector bundles |
This PR defines vector bundles (upstreamed from [formal-conjectures](https://github.com/google-deepmind/formal-conjectures/pull/28/files)). I plan on adding some more API about the definition in this PR, but figured it would be nice to get some initial feedback about the definition before doing so!
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
53/0 |
Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Sheaf/VectorBundle.lean |
2 |
2 |
['Kiolt', 'github-actions'] |
nobody |
0-36169 10 hours ago |
6-25847 6 days ago |
6-25893 6 days |
27271 |
ctchou author:ctchou |
feat: prove that each (total) preorder is an extension of a (linear) partial order |
Co-authored-by: Peter Nelson (original author)
---
This is a part of PR #27217, which continues the work in PR #12773.
[](https://gitpod.io/from-referrer/)
|
large-import
new-contributor
t-order
|
161/1 |
Mathlib/Order/Extension/Linear.lean,Mathlib/Order/Interval/Finset/Defs.lean,Mathlib/Order/RelClasses.lean |
3 |
4 |
['YaelDillies', 'b-mehta', 'ctchou', 'github-actions'] |
nobody |
0-35028 9 hours ago |
1-15069 1 day ago |
1-15117 1 day |
27278 |
artie2000 author:artie2000 |
feat: API for `Minpoly.toAdjoin` and friends |
* Replace `simps!` invocations on `AdjoinRoot.Minpoly.toAdjoin` and `minpoly.equivAdjoin` with principled API
* Create API for `AlgEquiv.adjoinSingletonEquivAdjoinRootMinpoly`
The auto-generated `simps!` lemmas unfolded the expressions too far for `simp` to be able to continue simplifying them. A good example of the difference is the proof of `Minpoly.toAdjoin.apply_X`.
---
[](https://gitpod.io/from-referrer/)
|
maintainer-merge
t-algebra
label:t-algebra$ |
24/14 |
Mathlib/FieldTheory/Minpoly/IsIntegrallyClosed.lean,Mathlib/RingTheory/Adjoin/Field.lean,Mathlib/RingTheory/AdjoinRoot.lean |
3 |
7 |
['YaelDillies', 'artie2000', 'github-actions'] |
nobody |
0-34351 9 hours ago |
0-34352 9 hours ago |
0-77351 21 hours |
27296 |
JovanGerb author:JovanGerb |
feat(Data/SetLike): `@[gcongr]` for `mem_of_le_of_mem` |
---
[](https://gitpod.io/from-referrer/)
|
t-data |
2/0 |
Mathlib/Data/SetLike/Basic.lean |
1 |
1 |
['github-actions'] |
nobody |
0-34322 9 hours ago |
0-34327 9 hours ago |
0-34383 9 hours |
27295 |
JovanGerb author:JovanGerb |
feat: `@[gcongr]` for `insert`/`erase` |
Also golf some proofs using these new tags. This also required tagging `adjoin.mono`.
---
[](https://gitpod.io/from-referrer/)
|
|
18/18 |
Archive/Imo/Imo2019Q2.lean,Mathlib/Data/Finset/Basic.lean,Mathlib/Data/Finset/Erase.lean,Mathlib/Data/Matroid/Circuit.lean,Mathlib/Data/Set/Insert.lean,Mathlib/FieldTheory/IntermediateField/Adjoin/Defs.lean,Mathlib/LinearAlgebra/AffineSpace/FiniteDimensional.lean,Mathlib/Topology/Algebra/Support.lean |
8 |
1 |
['github-actions'] |
nobody |
0-33820 9 hours ago |
0-39554 10 hours ago |
0-39536 10 hours |
27269 |
JovanGerb author:JovanGerb |
chore(Order/Monotone/Basic): rename `Monotone.eq_of_le_of_le` |
`Monotone.eq_of_ge_of_le` follows the new naming convention.
Also remove a duplicate of `lt_of_le_of_ne'`.
---
[](https://gitpod.io/from-referrer/)
|
|
8/7 |
Mathlib/Order/Monotone/Basic.lean,Mathlib/SetTheory/Ordinal/FixedPointApproximants.lean,Mathlib/Tactic/Linarith/Frontend.lean,Mathlib/Tactic/Positivity/Core.lean |
4 |
2 |
['JovanGerb', 'github-actions'] |
nobody |
0-32743 9 hours ago |
1-19723 1 day ago |
1-19705 1 day |
25943 |
101damnations author:101damnations |
feat(RepresentationTheory/Homological/GroupHomology): long exact sequences |
Given a commutative ring `k` and a group `G`, this PR shows that a short exact sequence of `k`-linear `G`-representations
`0 ⟶ X₁ ⟶ X₂ ⟶ X₃ ⟶ 0` induces a short exact sequence of complexes
`0 ⟶ inhomogeneousChains X₁ ⟶ inhomogeneousChains X₂ ⟶ inhomogeneousChains X₃ ⟶ 0`.
Since the homology of `inhomogeneousChains Xᵢ` is the group homology of `Xᵢ`, this allows us to specialize API about long exact sequences to group homology.
---
- [x] depends on: #21652
- [x] depends on: #21732
- [x] depends on: #21733
- [x] depends on: #21735
- [x] depends on: #21736
- [x] depends on: #21738
- [x] depends on: #25868
- [x] depends on: #25873
- [x] depends on: #25880
- [x] depends on: #25884
- [x] depends on: #25888
- [x] depends on: #25939
[](https://gitpod.io/from-referrer/)
---
*Earlier versions at #21764 and #21766*
|
t-algebra label:t-algebra$ |
514/4 |
Mathlib.lean,Mathlib/LinearAlgebra/Finsupp/Pi.lean,Mathlib/RepresentationTheory/Homological/GroupHomology/Basic.lean,Mathlib/RepresentationTheory/Homological/GroupHomology/Functoriality.lean,Mathlib/RepresentationTheory/Homological/GroupHomology/LongExactSequence.lean,Mathlib/RepresentationTheory/Homological/GroupHomology/LowDegree.lean,Mathlib/RepresentationTheory/Rep.lean |
7 |
n/a |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
0-32180 8 hours ago |
unknown |
unknown |
27292 |
gasparattila author:gasparattila |
feat: asymptotic cone of a set |
This PR defines the asymptotic cone of a set in a normed affine space and proves its main properties. This is partial progress towards showing that an unbounded finite-dimensional convex set contains a ray.
---
- [ ] depends on: #27221
[](https://gitpod.io/from-referrer/)
|
new-contributor |
441/0 |
Mathlib.lean,Mathlib/Analysis/Normed/Affine/AsymptoticCone.lean,Mathlib/Order/Filter/Map.lean |
3 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
0-32109 8 hours ago |
0-32110 8 hours ago |
0-33156 9 hours |
27243 |
artie2000 author:artie2000 |
chore(Algebra): add projection lemmas |
* Add `simp` projections for `Subsemiring.mk` by analogy with the same lemmas for other substructures.
* Add `simp` projection for `le` on `PartialOrder.mkOfGroupCone`.
Even though `PartialOrder.mkOfGroupCone` is an `abbrev`, the `simp` tactic cannot beta-reduce projections of class instances through `abbrev`s, so this additional `simp` lemma is necessary for the `LE` instance to be unfolded. See the discussion at https://leanprover.zulipchat.com/#narrow/channel/270676-lean4/topic/.60simp.60.20can't.20see.20through.20structure.20abbrevs.3F/with/525227013
---
[](https://gitpod.io/from-referrer/)
|
maintainer-merge
t-algebra
label:t-algebra$ |
24/1 |
Mathlib/Algebra/Order/Group/Cone.lean,Mathlib/Algebra/Order/Ring/Cone.lean,Mathlib/Algebra/Ring/Subsemiring/Defs.lean,Mathlib/FieldTheory/Fixed.lean |
4 |
24 |
['YaelDillies', 'artie2000', 'github-actions'] |
nobody |
0-29944 8 hours ago |
0-29944 8 hours ago |
1-50194 1 day |
26880 |
agjftucker author:agjftucker |
feat(Calculus/FDeriv/Partial): `hasStrictFDerivAt_uncurry_coprod` concerning partial derivatives |
Confident that other contributions will follow (e.g. #26300), I begin this file with only the result needed to apply the implicit function theorem to a curried function.
---
- [x] depends on: #26742 [This dependency is very slight.]
[](https://gitpod.io/from-referrer/)
|
new-contributor |
126/0 |
Mathlib.lean,Mathlib/Analysis/Calculus/FDeriv/Partial.lean |
2 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
0-29330 8 hours ago |
0-29330 8 hours ago |
4-20510 4 days |
27297 |
hugh-fox author:hugh-fox |
feat: add an equality between sums and products of cartesian products |
Adds `prod_mul_eq_prod_product` and a version for Finsets `prod_range_mul_eq_prod_product` with to show an equality between `Fin (i * j)` and `Fin a × Fin b`.
It is likely `prod_range_mul_eq_prod_product` belongs in a different file, in which case only the first commit should be considered.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-algebra
label:t-algebra$ |
18/0 |
Mathlib/Algebra/BigOperators/Fin.lean |
1 |
3 |
['github-actions', 'kckennylau'] |
nobody |
0-28645 7 hours ago |
0-29976 8 hours ago |
0-30021 8 hours |
27242 |
hugh-fox author:hugh-fox |
feat: add Gauss-like formula for sums of digit sums |
Adds `sum_digit_sum_base_pow_eq` to show a Gauss-like formula across sums of digit sums.
This relies on an additional two simp lemmas, named `digits_sum_eq_self`, `digits_sum_base_mul_cancel`.
Lastly, includes a specialization (which is a good bit simpler than the general formula) to base 10 named `sum_digit_sum_ten_pow_eq`.
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-data
new-contributor
|
113/0 |
Mathlib/Data/Nat/Digits/Lemmas.lean |
1 |
5 |
['github-actions', 'hugh-fox', 'kckennylau'] |
nobody |
0-28233 7 hours ago |
2-5611 2 days ago |
2-5657 2 days |
27216 |
D-Thomine author:D-Thomine |
feat(Cardinal/Finite): ENat powers and cardinality |
This PR continues the work from #25574.
Original PR: https://github.com/leanprover-community/mathlib4/pull/25574 |
t-algebra label:t-algebra$ |
172/3 |
Mathlib.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/Data/ENat/Pow.lean,Mathlib/SetTheory/Cardinal/Finite.lean |
4 |
8 |
['D-Thomine', 'eric-wieser', 'github-actions'] |
nobody |
0-26879 7 hours ago |
0-58049 16 hours ago |
1-75120 1 day |
26907 |
JovanGerb author:JovanGerb |
feat(gcongr): also use more general lemmas, closing extra goals with rfl |
This PR fixes an annoyance in tagging `gcongr` lemmas: if your function has `n` arguments in which to use congruence, then you would need to provide `2^n-1` `gcongr` lemmas. Now, it suffices to only tag the most general `gcongr` lemma, and in more specific cases, the extra goals will be closed using `rfl`.
While working on this, more issues with `gcongr` came up, and these all needed to be dealt with in the same PR:
- When applying a `gcongr` lemma, this should be done in the `reducible` transparency. The transparency was already bumped form `default` to `instances` after a zulip discussion ([#mathlib4 > gcongr unfold DFunLike.coe](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/gcongr.20unfold.20DFunLike.2Ecoe/with/482186693)). But I found that the same issue appears at `instances` transparency instead of `reducible`. MWE:
```
import Mathlib
open MeasureTheory
variable {α : Type*} (a : Set α) {μ : OuterMeasure α} {μ' : OuterMeasure α}
@[gcongr] -- remove this tag to make the last example work
lemma mono_outerMeasure (h : μ ≤ μ') : μ a ≤ μ' a := h a
example (h : μ ≤ μ') : μ a ≤ μ' a := by gcongr
variable [MeasurableSpace α] {ν : Measure α} {ν' : Measure α}
@[gcongr]
lemma mono_measure (h : ν ≤ ν') : ν a ≤ ν' a := h a
example (h : ν ≤ ν') : ν a ≤ ν' a := by
with_reducible apply mono_outerMeasure
set_option trace.Meta.isDefEq true in
with_reducible gcongr
```
This aligns with the `congr!` tactic
- Using `reducible` transparency is not compatible with the approach of matching `varyingArgs`, because when comparing instance arguments, we need to use at least `instances` transparency. So, instead of storing the lemmas by `varyingArgs`, we sort them by the number of varying arguments, and simply try applying all the lemmas (which should be cheap in `reducible` transparency). This aligns with `congr`/`congr!`(/`simp`) which also tries all of the lemmas for the given constant.
- As a result of sorting the lemmas in the same way as `congr` lemmas, more recently added lemmas are now tried before older ones. This causes an issue which has to be solved by implementing a priority argument for the `gcongr` tag (similar to how `instance` and `simp` work), e.g.`@[gcongr high]`. This aligns with the `@[congr]` tag.
---
[](https://gitpod.io/from-referrer/)
|
|
330/293 |
Mathlib/Algebra/Group/Pointwise/Finset/Basic.lean,Mathlib/Algebra/Group/Pointwise/Set/Basic.lean,Mathlib/Algebra/Group/Pointwise/Set/Scalar.lean,Mathlib/Algebra/Order/GroupWithZero/Unbundled/Basic.lean,Mathlib/Algebra/Order/Monoid/Unbundled/Basic.lean,Mathlib/Algebra/Order/Sub/Defs.lean,Mathlib/Algebra/Ring/Submonoid/Pointwise.lean,Mathlib/Analysis/Complex/UpperHalfPlane/Topology.lean,Mathlib/Analysis/Distribution/SchwartzSpace.lean,Mathlib/Analysis/FunctionalSpaces/SobolevInequality.lean,Mathlib/Analysis/MellinTransform.lean,Mathlib/Combinatorics/SimpleGraph/Subgraph.lean,Mathlib/Data/ENNReal/Inv.lean,Mathlib/Data/Finset/Lattice/Basic.lean,Mathlib/Data/Finset/NAry.lean,Mathlib/Data/Finset/Prod.lean,Mathlib/Data/Int/ModEq.lean,Mathlib/Data/List/Perm/Basic.lean,Mathlib/Data/Nat/Basic.lean,Mathlib/Data/Nat/ModEq.lean,Mathlib/Data/Set/Basic.lean,Mathlib/Data/Set/NAry.lean,Mathlib/Data/Set/Prod.lean,Mathlib/MeasureTheory/Function/LpSeminorm/Basic.lean,Mathlib/MeasureTheory/Function/SimpleFunc.lean,Mathlib/MeasureTheory/Integral/Lebesgue/Basic.lean,Mathlib/MeasureTheory/Measure/Lebesgue/EqHaar.lean,Mathlib/MeasureTheory/Measure/Restrict.lean,Mathlib/NumberTheory/Bertrand.lean,Mathlib/Order/Basic.lean,Mathlib/Order/BooleanAlgebra/Set.lean,Mathlib/Order/Disjoint.lean,Mathlib/Order/Filter/NAry.lean,Mathlib/Order/Filter/Prod.lean,Mathlib/Order/Fin/Basic.lean,Mathlib/Order/Heyting/Basic.lean,Mathlib/Order/Interval/Finset/Basic.lean,Mathlib/Order/Interval/Set/Basic.lean,Mathlib/Order/Lattice.lean,Mathlib/Order/RelClasses.lean,Mathlib/Order/Sublattice.lean,Mathlib/RingTheory/Ideal/Prod.lean,Mathlib/Tactic/GCongr/Core.lean,Mathlib/Tactic/GCongr/CoreAttrs.lean,Mathlib/Tactic/Monotonicity/Lemmas.lean,Mathlib/Topology/UniformSpace/Defs.lean,MathlibTest/GCongr/GCongr.lean,MathlibTest/GCongr/implications.lean,MathlibTest/GCongr/inequalities.lean,MathlibTest/GRewrite.lean |
50 |
14 |
['JovanGerb', 'Vtec234', 'fpvandoorn', 'github-actions', 'grunweg'] |
nobody |
0-26865 7 hours ago |
9-14967 9 days ago |
10-8384 10 days |
26843 |
vasnesterov author:vasnesterov |
feat(Tactic/Simproc): nested quantifiers in `existsAndEq` |
Generalize the `existsAndEq` simproc to nested existential quantifiers.
For example `∃ a, p a ∧ ∃ b, a = f b ∧ q b` now simplifies to `∃ b, p (f b) ∧ q b`.
---
[](https://gitpod.io/from-referrer/)
This PR continues the work from #23365.
Original PR: https://github.com/leanprover-community/mathlib4/pull/23365 |
migrated-from-branch
large-import
t-meta
|
452/79 |
Mathlib/Data/List/ProdSigma.lean,Mathlib/Tactic/Simproc/ExistsAndEq.lean,MathlibTest/Simproc/ExistsAndEq.lean |
3 |
7 |
['JovanGerb', 'github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'vasnesterov'] |
nobody |
0-26324 7 hours ago |
12-56641 12 days ago |
12-70692 12 days |
25864 |
plp127 author:plp127 |
feat(Nat/Digits): use fuel in `Nat.digits` |
Add a `fuel` parameter to `Nat.digitsAux` to make it structurally recursive.
---
[](https://gitpod.io/from-referrer/)
|
t-data |
47/14 |
Mathlib/Data/Nat/Digits/Defs.lean |
1 |
2 |
['github-actions', 'leanprover-community-bot-assistant'] |
nobody |
0-19507 5 hours ago |
0-21538 5 hours ago |
20-68096 20 days |
27299 |
alreadydone author:alreadydone |
chore(EllipticCurve): make affine addition computable |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-algebraic-geometry
label:t-algebra$ |
108/78 |
Mathlib/AlgebraicGeometry/EllipticCurve/Affine/Formula.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Affine/Point.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Jacobian/Formula.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Jacobian/Point.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Projective/Formula.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Projective/Point.lean |
6 |
1 |
['github-actions'] |
nobody |
0-18481 5 hours ago |
0-18565 5 hours ago |
0-18548 5 hours |
25945 |
adomani author:adomani |
feat: the empty line in commands linter |
This linter flags empty lines within a command.
It allows empty lines within doc-strings, module-docs and a couple of other "sensible" places.
It also skips files that are likely to contain meta-code, since there the use of empty lines in definition is more widespread.
This PR continues the work from #25236. |
large-import
maintainer-merge
|
375/7 |
Mathlib.lean,Mathlib/Analysis/Meromorphic/FactorizedRational.lean,Mathlib/CategoryTheory/Comma/StructuredArrow/CommaMap.lean,Mathlib/Init.lean,Mathlib/RepresentationTheory/Homological/GroupHomology/LowDegree.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter/EmptyLine.lean,MathlibTest/EmptyLine.lean |
8 |
3 |
['adomani', 'github-actions'] |
bryangingechen assignee:bryangingechen |
0-17530 4 hours ago |
33-75531 1 month ago |
33-75584 33 days |
27301 |
js2357 author:js2357 |
feat: `MeasureTheory.Measure.sum_restrict_le` |
Prove that `Measure.sum (fun i ↦ μ.restrict (s i)) ≤ M • μ.restrict (⋃ i, s i)`, if at most `M` of the `s i` overlap at a single point.
Also add `restrict_biUnion_le`, which is a straightforward biUnion version of the existing `restrict_iUnion_le`.
Done for the Carleson project.
[](https://gitpod.io/from-referrer/)
|
carleson
t-measure-probability
|
87/0 |
Mathlib.lean,Mathlib/MeasureTheory/Measure/Restrict.lean,Mathlib/MeasureTheory/Measure/SumRestrict.lean |
3 |
1 |
['github-actions'] |
nobody |
0-14289 3 hours ago |
0-14296 3 hours ago |
0-14342 3 hours |
27282 |
artie2000 author:artie2000 |
feat(Algebra/Order/Ring): define ring orderings |
Define preorderings, their supports, orderings
These objects are the right generalisation of the "positive cones" / "orderings" defined on fields in the classical Artin-Schreier argument that a field can be ordered if and only if -1 is not a sum of squares. See *An introduction to real algebra* by T.Y. Lam for details.
Contrast `Algebra.Order.Ring.Cone`, which defines an algebraic axiomatisation of a (partially/linearly) ordered ring.
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebra
label:t-algebra$ |
218/20 |
Mathlib.lean,Mathlib/Algebra/Group/Subgroup/Defs.lean,Mathlib/Algebra/Order/Group/Cone.lean,Mathlib/Algebra/Order/Ring/Cone.lean,Mathlib/Algebra/Order/Ring/Ordering/Defs.lean |
5 |
34 |
['YaelDillies', 'artie2000', 'github-actions'] |
nobody |
0-10172 2 hours ago |
0-23112 6 hours ago |
0-58267 16 hours |