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 |
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 |
90-19067 2 months ago |
159-20709 5 months ago |
159-20831 159 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 |
85-71877 2 months ago |
106-44321 3 months ago |
117-6735 117 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 |
82-47041 2 months ago |
82-52992 2 months ago |
130-18810 130 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 |
82-17034 2 months ago |
82-17034 2 months ago |
105-41151 105 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 |
81-7149 2 months ago |
81-15789 2 months ago |
81-15840 81 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 |
75-84502 2 months ago |
91-84142 2 months ago |
92-5654 92 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 |
74-55298 2 months ago |
74-55422 2 months ago |
74-58884 74 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 |
72-27519 2 months ago |
100-25076 3 months ago |
100-25127 100 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 |
67-56211 2 months ago |
109-44509 3 months ago |
109-44558 109 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 |
67-46666 2 months ago |
73-23067 2 months ago |
73-23062 73 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 |
66-7539 2 months ago |
69-59678 2 months ago |
69-59659 69 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 |
64-52728 2 months ago |
64-52728 2 months ago |
64-71110 64 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 |
61-21391 2 months ago |
62-31113 2 months ago |
62-31101 62 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 |
53-15243 1 month ago |
53-15306 1 month ago |
68-47241 68 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 |
50-70127 1 month ago |
50-76826 1 month ago |
50-76809 50 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 |
50-66924 1 month ago |
51-17393 1 month ago |
51-17375 51 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 |
49-63891 1 month ago |
49-63891 1 month ago |
49-69024 49 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 |
45-82451 1 month ago |
45-82451 1 month ago |
45-84976 45 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 |
44-83579 1 month ago |
68-48140 2 months ago |
68-52061 68 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 |
44-39250 1 month ago |
48-71049 1 month ago |
48-71093 48 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 |
43-72560 1 month ago |
43-72560 1 month ago |
43-72619 43 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 |
43-68162 1 month ago |
43-68323 1 month ago |
43-68376 43 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 |
42-84124 1 month ago |
42-84130 1 month ago |
42-84175 42 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 |
42-42782 1 month ago |
44-13673 1 month ago |
44-13655 44 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 |
42-36938 1 month ago |
42-36938 1 month ago |
42-41550 42 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 |
41-48443 1 month ago |
45-29707 1 month ago |
45-29753 45 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 |
40-65556 1 month ago |
44-46892 1 month ago |
44-46942 44 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 |
40-15140 1 month ago |
40-15163 1 month ago |
40-29079 40 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 |
39-68930 1 month ago |
39-68940 1 month ago |
39-68984 39 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 |
39-59400 1 month ago |
39-59401 1 month ago |
43-29002 43 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 |
39-20585 1 month ago |
39-20592 1 month ago |
39-20635 39 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 |
33-66355 1 month ago |
33-66381 1 month ago |
33-66426 33 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 |
32-70683 1 month ago |
42-3863 1 month ago |
49-35248 49 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 |
32-66164 1 month ago |
38-69548 1 month ago |
38-69599 38 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 |
32-28964 1 month ago |
46-79791 1 month ago |
47-1992 47 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 |
30-35605 30 days ago |
30-35784 30 days ago |
30-75206 30 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 |
30-29287 30 days ago |
32-42143 1 month ago |
111-18681 111 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 |
30-6421 30 days ago |
30-6421 30 days ago |
43-78340 43 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 |
29-67713 29 days ago |
107-81096 3 months ago |
163-41815 163 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 |
29-57917 29 days ago |
39-59438 1 month ago |
39-59489 39 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 |
29-42550 29 days ago |
35-27038 1 month ago |
51-82841 51 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 |
29-33811 29 days ago |
29-62316 29 days ago |
29-62368 29 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 |
29-31234 29 days ago |
29-31365 29 days ago |
29-31417 29 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 |
29-12102 29 days ago |
30-396 30 days ago |
43-2984 43 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 |
29-10647 29 days ago |
29-20143 29 days ago |
29-26457 29 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 |
28-48041 28 days ago |
28-48041 28 days ago |
28-48024 28 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 |
28-6883 28 days ago |
28-9465 28 days ago |
182-46795 182 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 |
28-6711 28 days ago |
28-6729 28 days ago |
50-82314 50 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 |
28-6246 28 days ago |
28-6268 28 days ago |
144-83287 144 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 |
28-5681 28 days ago |
28-10961 28 days ago |
44-57011 44 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 |
28-3751 28 days ago |
31-18519 1 month ago |
31-19077 31 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 |
28-3470 28 days ago |
44-46845 1 month ago |
45-23300 45 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 |
28-3170 28 days ago |
28-3215 28 days ago |
49-47983 49 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 |
27-43932 27 days ago |
27-47114 27 days ago |
149-83917 149 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 |
27-4360 27 days ago |
27-83929 27 days ago |
28-576 28 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 |
26-85455 26 days ago |
82-70644 2 months ago |
84-20470 84 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 |
26-82922 26 days ago |
26-82922 26 days ago |
28-66486 28 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 |
26-65913 26 days ago |
31-24069 1 month ago |
31-24114 31 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 |
26-50644 26 days ago |
28-39458 28 days ago |
28-39502 28 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 |
26-30431 26 days ago |
26-54071 26 days ago |
26-54054 26 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 |
25-79210 25 days ago |
26-26782 26 days ago |
49-6958 49 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 |
23-85501 23 days ago |
25-52087 25 days ago |
47-55756 47 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 |
23-10435 23 days ago |
26-85804 26 days ago |
26-85849 26 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 |
22-48716 22 days ago |
25-45754 25 days ago |
25-45798 25 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 |
22-35084 22 days ago |
45-75151 1 month ago |
45-75200 45 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 |
21-76325 21 days ago |
21-80150 21 days ago |
21-80201 21 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 |
21-67116 21 days ago |
21-67118 21 days ago |
21-67170 21 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 |
21-12772 21 days ago |
21-13074 21 days ago |
21-13058 21 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 |
21-2616 21 days ago |
26-5125 26 days ago |
26-5179 26 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 |
20-65512 20 days ago |
20-67135 20 days ago |
20-67130 20 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 |
20-47693 20 days ago |
20-47702 20 days ago |
20-47747 20 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 |
19-70756 19 days ago |
19-82664 19 days ago |
19-84364 19 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 |
19-34170 19 days ago |
20-36662 20 days ago |
20-36882 20 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 |
19-31878 19 days ago |
19-31894 19 days ago |
19-61446 19 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 |
19-16622 19 days ago |
19-16625 19 days ago |
19-16679 19 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 |
19-10250 19 days ago |
50-66578 1 month ago |
50-66561 50 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 |
18-73911 18 days ago |
22-79533 22 days ago |
22-79583 22 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 |
18-69902 18 days ago |
20-7927 20 days ago |
20-7910 20 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 |
18-64210 18 days ago |
21-62437 21 days ago |
21-62420 21 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 |
18-63626 18 days ago |
18-63626 18 days ago |
18-73417 18 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 |
18-59968 18 days ago |
19-14972 19 days ago |
19-14966 19 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 |
18-59033 18 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 |
18-56426 18 days ago |
19-9527 19 days ago |
19-9570 19 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 |
17-80441 17 days ago |
27-46832 27 days ago |
135-26361 135 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 |
17-60117 17 days ago |
17-60141 17 days ago |
179-48098 179 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 |
17-59635 17 days ago |
17-79833 17 days ago |
73-63101 73 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 |
17-33290 17 days ago |
19-67831 19 days ago |
19-67872 19 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 |
17-22953 17 days ago |
26-27016 26 days ago |
49-9404 49 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 |
16-68851 16 days ago |
16-68852 16 days ago |
16-69166 16 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 |
16-67438 16 days ago |
16-67789 16 days ago |
16-67933 16 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 |
16-57617 16 days ago |
17-36180 17 days ago |
17-36222 17 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 |
16-26067 16 days ago |
16-27486 16 days ago |
16-27543 16 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 |
16-14702 16 days ago |
17-73183 17 days ago |
20-65934 20 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 |
15-64717 15 days ago |
21-1246 21 days ago |
21-1319 21 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 |
15-47649 15 days ago |
17-42574 17 days ago |
17-42618 17 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 |
15-31561 15 days ago |
26-35350 26 days ago |
26-36067 26 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 |
15-28435 15 days ago |
17-67303 17 days ago |
17-67910 17 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 |
15-6931 15 days ago |
51-47876 1 month ago |
112-33598 112 days |
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 |
14-83864 14 days ago |
14-83882 14 days ago |
45-332 45 days |
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 |
14-69632 14 days ago |
17-18 17 days ago |
17-10462 17 days |
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 |
14-62745 14 days ago |
15-2834 15 days ago |
15-2878 15 days |
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 |
14-48635 14 days ago |
15-52113 15 days ago |
15-56430 15 days |
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 |
14-41768 14 days ago |
14-52399 14 days ago |
14-52447 14 days |
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 |
14-40617 14 days ago |
14-40627 14 days ago |
14-40672 14 days |
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 |
14-40613 14 days ago |
14-40617 14 days ago |
14-40661 14 days |
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 |
14-39048 14 days ago |
14-39181 14 days ago |
49-73339 49 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 |
14-23517 14 days ago |
35-20835 1 month ago |
35-25587 35 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 |
14-20982 14 days ago |
14-21002 14 days ago |
36-27985 36 days |
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 |
13-69625 13 days ago |
38-49011 1 month ago |
38-49058 38 days |
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 |
13-45627 13 days ago |
13-45627 13 days ago |
17-36807 17 days |
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 |
13-44530 13 days ago |
15-21908 15 days ago |
15-21955 15 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$ |
204/5 |
Mathlib.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/Data/ENat/Pow.lean,Mathlib/SetTheory/Cardinal/Finite.lean |
4 |
12 |
['D-Thomine', 'eric-wieser', 'github-actions'] |
nobody |
12-71434 12 days ago |
13-74346 13 days ago |
15-5018 15 days |
27312 |
pechersky author:pechersky |
feat(RingTheory/Valuation): the trivial valuation, as One (Valuation R Γ₀) |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-number-theory
label:t-algebra$ |
54/0 |
Mathlib/Algebra/GroupWithZero/Hom.lean,Mathlib/RingTheory/Valuation/Basic.lean |
2 |
1 |
['github-actions'] |
nobody |
12-46539 12 days ago |
12-46601 12 days ago |
12-46594 12 days |
24530 |
chrisflav author:chrisflav |
feat(RingTheory): faithfully flat ring maps |
Co-authored by: Joël Riou
---
- [x] depends on: #24375
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
89/1 |
Mathlib.lean,Mathlib/Algebra/Ring/Equiv.lean,Mathlib/RingTheory/RingHom/FaithfullyFlat.lean,Mathlib/RingTheory/RingHom/Flat.lean |
4 |
7 |
['chrisflav', 'erdOne', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
12-12522 12 days ago |
12-70094 12 days ago |
68-50071 68 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-55598 11 days ago |
44-58754 1 month ago |
44-58757 44 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 |
11-20839 11 days ago |
19-56653 19 days ago |
19-56698 19 days |
27357 |
jcreedcmu author:jcreedcmu |
feat(Algebra/Module/Submodule): add `submoduleMap` for isometries |
Per [discussion on Zulip](https://leanprover.zulipchat.com/#narrow/channel/217875-Is-there-code-for-X.3F/topic/Analog.20of.20LinearEquiv.2EsubmoduleMap.20for.20AffineIsometryEquiv.3F), add a version of `.submoduleMap` for `LinearIsometry` and `LinearIsometryEquiv` by analogy with `LinearMap.submoduleMap` and `LinearEquiv.submoduleMap`.
--- |
new-contributor
t-algebra
label:t-algebra$ |
56/0 |
Mathlib.lean,Mathlib/Analysis/Normed/Operator/LinearIsometrySubmoduleMap.lean |
2 |
12 |
['Ruben-VandeVelde', 'eric-wieser', 'github-actions', 'jcreedcmu'] |
nobody |
10-38622 10 days ago |
10-43805 10 days ago |
10-43857 10 days |
27370 |
euprunin author:euprunin |
chore(Tactic/CancelDenoms): golf `cancel_factors_eq` |
|
t-meta |
1/11 |
Mathlib/Tactic/CancelDenoms/Core.lean |
1 |
1 |
['github-actions'] |
nobody |
10-34443 10 days ago |
10-34462 10 days ago |
10-34511 10 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 |
13 |
['YaelDillies', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'robin-carlier', 'yuma-mizuno'] |
nobody |
10-5523 10 days ago |
10-5542 10 days ago |
33-69669 33 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/73 |
Mathlib.lean,Mathlib/RingTheory/OreLocalization/Basic.lean,Mathlib/RingTheory/OreLocalization/NonZeroDivisors.lean,Mathlib/RingTheory/OreLocalization/Ring.lean |
4 |
2 |
['github-actions', 'leanprover-community-bot-assistant'] |
nobody |
10-796 10 days ago |
10-1253 10 days ago |
17-29823 17 days |
26847 |
joelriou author:joelriou |
feat: multicoequalizers in the category of types |
This PR gives a concrete criteria for a multicofork in the category of types to be a multicoequalizer, and this is used in order to show that if a (sub)set `A : Set X` is the union of certain subsets `U i`, then the type `A` is the multicoequalizer of the `U i`s along their intersections `V i j`.
(A similar result for `Subpresheaf` rather than `Set` will be deduced in a separate PR, and this shall be very important in the study of the homotopy theory of simplicial sets, as this will allow the construction of morphisms from horns.)
---
- [x] depends on: #25823
- [x] depends on: #22205
- [x] depends on: #26037
This PR continues the work from #23872.
Original PR: https://github.com/leanprover-community/mathlib4/pull/23872 |
t-category-theory |
96/0 |
Mathlib.lean,Mathlib/CategoryTheory/Limits/Types/Multicoequalizer.lean |
2 |
n/a |
['adomani', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
9-75934 9 days 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 |
6 |
['YaelDillies', 'artie2000', 'eric-wieser', 'github-actions'] |
nobody |
9-36708 9 days ago |
14-20142 14 days ago |
14-22362 14 days |
27417 |
PierreQuinton author:PierreQuinton |
feat: add `SigmaCompleteLattice` |
A $\sigma$-complete lattice is a lattice in which every countable subset `s` has a least upper bound and a greatest lower bound, denoted below by `sSup s` and `sInf s`.
This PR adds the classes `SigmaCompleteLattice` as well as some theorems (mainly adapted from `CompleteLattice` and `ConditionallyCompleteLattice`). This is an adaptation of #26318
---
[](https://gitpod.io/from-referrer/)
|
t-order |
394/0 |
Mathlib.lean,Mathlib/Order/SigmaCompleteLattice.lean |
2 |
3 |
['PierreQuinton', 'github-actions', 'vihdzp'] |
nobody |
8-79753 8 days ago |
9-4891 9 days ago |
9-4939 9 days |
27427 |
alreadydone author:alreadydone |
chore(RingTheory): use `extend` instead of `abbrev` in `IsS(emis)impleModule` |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
46/37 |
Mathlib/Algebra/Category/ModuleCat/Simple.lean,Mathlib/Algebra/Module/PID.lean,Mathlib/LinearAlgebra/RootSystem/Irreducible.lean,Mathlib/LinearAlgebra/Semisimple.lean,Mathlib/RepresentationTheory/Maschke.lean,Mathlib/RingTheory/Length.lean,Mathlib/RingTheory/SimpleModule/Basic.lean,Mathlib/RingTheory/SimpleModule/Rank.lean |
8 |
4 |
['alreadydone', 'github-actions', 'leanprover-bot'] |
nobody |
8-48000 8 days ago |
8-48000 8 days ago |
8-47984 8 days |
27453 |
pechersky author:pechersky |
feat(Topology/UniformSpace/Ultra): completion is ultra uniformity iff base is |
Supersedes #24628
---
[](https://gitpod.io/from-referrer/)
|
t-topology |
159/5 |
Mathlib.lean,Mathlib/Order/Filter/NAry.lean,Mathlib/Order/Filter/Prod.lean,Mathlib/Topology/Constructions/SumProd.lean,Mathlib/Topology/UniformSpace/Defs.lean,Mathlib/Topology/UniformSpace/Ultra/Basic.lean,Mathlib/Topology/UniformSpace/Ultra/Completion.lean |
7 |
1 |
['github-actions'] |
nobody |
8-28132 8 days ago |
8-28192 8 days ago |
8-28187 8 days |
27455 |
pechersky author:pechersky |
chore(NumberTheory/Padics/Hensel): rephrase using `aeval` |
This is easier to use at call site, because on need not pass `Polynomial.map (algebraMap _ _ )` in the use of `hensels_lemma`
---
[](https://gitpod.io/from-referrer/)
|
tech debt
t-algebra
t-number-theory
label:t-algebra$ |
157/138 |
Mathlib/NumberTheory/Padics/Hensel.lean |
1 |
1 |
['github-actions'] |
nobody |
8-21974 8 days ago |
8-22029 8 days ago |
8-22027 8 days |
27460 |
IvanRenison author:IvanRenison |
feat(Combinatorics/SimpleGraph/Walk): add theorems about membership on the support of `Walk.concat` |
This contribution was created as part of the Utrecht Summerschool "Formalizing Mathematics in Lean" in July 2025.
---
[](https://gitpod.io/from-referrer/)
|
t-combinatorics |
18/0 |
Mathlib/Combinatorics/SimpleGraph/Walk.lean |
1 |
1 |
['github-actions'] |
nobody |
7-70551 7 days ago |
7-82152 7 days ago |
7-82194 7 days |
27464 |
IvanRenison author:IvanRenison |
feat(Combinatorics/SimpleGraph/Paths): add lemma `SimpleGraph.Walk.IsPath.ne_of_mem_support_of_append` |
This contribution was created as part of the Utrecht Summerschool "Formalizing Mathematics in Lean" in July 2025.
---
[](https://gitpod.io/from-referrer/)
|
t-combinatorics |
7/0 |
Mathlib/Combinatorics/SimpleGraph/Paths.lean |
1 |
1 |
['github-actions'] |
nobody |
7-70535 7 days ago |
7-79867 7 days ago |
7-79917 7 days |
27468 |
IvanRenison author:IvanRenison |
feat(Combinatorics/SimpleGraph): add theorem `SimpleGraph.Connected.diff_dist_adj` |
This contribution was created as part of the Utrecht Summerschool "Formalizing Mathematics in Lean" in July 2025.
---
[](https://gitpod.io/from-referrer/)
|
t-combinatorics |
16/0 |
Mathlib/Combinatorics/SimpleGraph/Metric.lean |
1 |
1 |
['github-actions'] |
nobody |
7-70529 7 days ago |
7-72050 7 days ago |
7-72149 7 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$ |
469/67 |
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 |
5 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
7-69833 7 days ago |
7-69982 7 days ago |
76-28523 76 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 |
364/1 |
Mathlib/CategoryTheory/Limits/Shapes/Pullback/Categorical/Basic.lean |
1 |
4 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'robin-carlier'] |
nobody |
7-64410 7 days ago |
7-64410 7 days ago |
17-11652 17 days |
27447 |
eric-wieser author:eric-wieser |
refactor: rename `Rel` to `Set.Rel`, restore the old `Rel` |
Many users are confused that Rel no longer means what it used to. Since the design is not obvious, let's put it in a namespace that makes the choice obvious.
This then restores the old definition of `Rel`, as an abbrev; it's conceivable that many users were just using this as a shorthand, and this stops them being broken by #25587. Such users will of course be broken if they used [the old API](https://github.com/leanprover-community/mathlib4/blob/59bd63c72671849996d64c5d3b5f24a36333483c%5E/Mathlib/Data/Rel.lean).
This way, users bumping from 4.21.0 to 4.22.0 and using `Rel` only as a shorthand will not be broken.
[#mathlib4 > Changing `Rel` to `Set (α × β)`, to help uniform spaces @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Changing.20.60Rel.60.20to.20.60Set.20.28.CE.B1.20.C3.97.20.CE.B2.29.60.2C.20to.20help.20uniform.20spaces/near/528531852)
---
[](https://gitpod.io/from-referrer/)
|
t-order |
134/116 |
Mathlib/CategoryTheory/Category/RelCat.lean,Mathlib/Combinatorics/Hall/Basic.lean,Mathlib/Combinatorics/SimpleGraph/Basic.lean,Mathlib/Combinatorics/SimpleGraph/Subgraph.lean,Mathlib/Data/PFun.lean,Mathlib/Data/Rel.lean,Mathlib/Order/Filter/Partial.lean,Mathlib/Order/KrullDimension.lean,Mathlib/Order/Rel/GaloisConnection.lean,Mathlib/Order/RelSeries.lean,Mathlib/RingTheory/Length.lean,Mathlib/Topology/Partial.lean,Mathlib/Topology/UniformSpace/Basic.lean |
13 |
3 |
['YaelDillies', 'eric-wieser', 'github-actions'] |
nobody |
7-64370 7 days ago |
7-80502 7 days ago |
8-34455 8 days |
25951 |
themathqueen author:themathqueen |
feat(Analysis/InnerProductSpace/MulOpposite): defines the inner product on opposite spaces |
This pr defines the inner product on opposite spaces.
- [x] depends on: #25949
Motivation for having the inner product structure on the opposite:
One application comes up in non-commutative graphs, which are defined on a finite-dimensional C*-algebra with a faithful and positive functional (a Hilbert space structure can be induced by the defined faithful and positive functional (will be added to a pr soon)). For example, we'd need the Hilbert space structure to be defined on the opposite space to define the isomorphism: `(A →ₗ[ℂ] B) ≃ₗ[ℂ] TensorProduct ℂ B Aᵐᵒᵖ`, where `A`, `B` are again finite-dimensional C*-algebras with faithful and positive functionals.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor |
71/0 |
Mathlib.lean,Mathlib/Analysis/InnerProductSpace/MulOpposite.lean |
2 |
6 |
['github-actions', 'j-loreaux', 'mathlib4-dependent-issues-bot', 'themathqueen'] |
nobody |
7-58868 7 days ago |
9-76276 9 days ago |
27-11387 27 days |
27441 |
judithludwig author:judithludwig |
feat(RingTheory/Polynomial/Quotient): Lemma on PIDs |
This is part of a course project at Heidelberg University: https://matematiflo.github.io/CompAssistedMath2025/
feat(RingTheory/Polynomial/Quotient): add lemma: Let $$R$$ be an integral domain and assume $$R[X]$$ is a PID, then $$R$$ is a field. This lemma is useful for proving that some rings are not PIDs, such as $$\mathbb{Z}[X]$$.
Co-authored-by: Philipp Sivov @Silipp182
Co-authored-by: Veliyan Taslev @hubavelko
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
11/0 |
Mathlib/RingTheory/Polynomial/Quotient.lean |
1 |
3 |
['alreadydone', 'github-actions'] |
nobody |
7-55126 7 days ago |
8-46112 8 days ago |
8-46158 8 days |
26912 |
pechersky author:pechersky |
chore(Algebra/Ring/Subring): simp tag `Subring.smul_def` |
s-multiplying by a subtype is easiest to manipulate when both terms are in the ambient type. Many places that had to use the _def lemma for a rewrite, or to include it in a simp set, no longer have to.
Ported from #25308
---
[](https://gitpod.io/from-referrer/)
I found this being not-simp frustrating when talking about submodules over a valuation subring. |
maintainer-merge
t-algebra
label:t-algebra$ |
68/67 |
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/Exact.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/Etale/Kaehler.lean,Mathlib/RingTheory/LocalProperties/Projective.lean,Mathlib/RingTheory/Localization/InvSubmonoid.lean,Mathlib/RingTheory/OreLocalization/Basic.lean |
25 |
16 |
['eric-wieser', 'github-actions', 'j-loreaux', 'linesthatinterlace', 'pechersky'] |
nobody |
7-49782 7 days ago |
10-42672 10 days ago |
21-57546 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 |
5 |
['adomani', 'github-actions', 'grunweg', 'leanprover-bot'] |
nobody |
7-36671 7 days ago |
39-68255 1 month ago |
39-72887 39 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$ |
150/13 |
Mathlib/Algebra/Algebra/Tower.lean,Mathlib/RingTheory/Ideal/Norm/RelNorm.lean,Mathlib/RingTheory/Ideal/Prime.lean,Mathlib/RingTheory/IntegralClosure/IntegralRestrict.lean,Mathlib/RingTheory/Localization/AtPrime.lean,Mathlib/RingTheory/Localization/FractionRing.lean |
6 |
5 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'riccardobrasca', 'xroblot'] |
riccardobrasca assignee:riccardobrasca |
7-33366 7 days ago |
17-35068 17 days ago |
17-46016 17 days |
25182 |
YaelDillies author:YaelDillies |
feat: `(M →* N₁) ≃* (M →* N₂)` if `N₁ ≃* N₂` |
The names were discussed on [Zulip](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Naming.20congruence.20of.20maps) but no consensus was reached due to lack of engagement.
The names I choose here are consistent with [`ContinuousLinearEquiv.continuousAlternatingMapCongrLeft`](https://leanprover-community.github.io/mathlib4_docs/find/?pattern=ContinuousLinearEquiv.continuousAlternatingMapCongrLeft#doc) and around.
From Toric
---
[](https://gitpod.io/from-referrer/)
|
toric
t-algebra
label:t-algebra$ |
116/18 |
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 |
20 |
['YaelDillies', 'b-mehta', 'eric-wieser', 'github-actions'] |
eric-wieser assignee:eric-wieser |
7-4233 7 days ago |
8-59850 8 days ago |
66-51111 66 days |
27497 |
ScottCarnahan author:ScottCarnahan |
feat(RingTheory/PowerSeries/Binomial): add basic lemmas, golf |
This PR adds two simp lemmas for binomial power series, and generalizes the hypotheses of `binomialSeries_nat`.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
17/19 |
Mathlib/RingTheory/PowerSeries/Binomial.lean |
1 |
3 |
['ScottCarnahan', 'github-actions', 'wwylele'] |
nobody |
6-79767 6 days ago |
7-30172 7 days ago |
7-30167 7 days |
27498 |
Komyyy author:Komyyy |
feat: Group isomorphisms between (`Equiv.Perm`|`alternatingGroup`)s |
Required to prove that A_n is simple iff n = 3 or 5 ≤ n(#26051).
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
29/0 |
Mathlib/Algebra/Group/End.lean,Mathlib/GroupTheory/SpecificGroups/Alternating.lean |
2 |
1 |
['github-actions'] |
nobody |
6-56862 6 days ago |
7-29617 7 days ago |
7-29602 7 days |
27516 |
gaetanserre author:gaetanserre |
feat: add rational approximation lemma for suprema in `unitInterval` |
Add `sSup_eq_iUnion_rat` lemma that provides a rational approximation characterization of suprema in the unit interval. For monotone functions `f : α → I → ℝ`, the lemma establishes that the set of pairs where `a < sSup {x | f e.1 x < e.2}` equals the union over all rationals `q ∈ I` with `q > a` of the sets `{e | f e.1 q < e.2}`.
---
[](https://gitpod.io/from-referrer/)
|
t-topology |
21/0 |
Mathlib/Topology/UnitInterval.lean |
1 |
1 |
['github-actions'] |
nobody |
6-52318 6 days ago |
6-56397 6 days ago |
6-56442 6 days |
27515 |
gaetanserre author:gaetanserre |
feat: `ProbabilityTheory.cdf_eq_real` for measure on `unitInterval` |
Given a probability measure `μ` on `I`, the CDF of the pushforward of `μ` along `Subtype.val` is equal to the measure of the closed interval.
---
[](https://gitpod.io/from-referrer/)
|
t-measure-probability |
9/0 |
Mathlib/Probability/CDF.lean |
1 |
1 |
['github-actions'] |
nobody |
6-52295 6 days ago |
6-57961 6 days ago |
6-58006 6 days |
27517 |
gaetanserre author:gaetanserre |
feat: a `MeasurableEmbedding` has a measurable left inverse |
Definition of the measurable left inverse of a `MeasurableEmbedding`.
Co-authored-by: Rémy Degenne
---
[](https://gitpod.io/from-referrer/)
|
t-measure-probability |
29/0 |
Mathlib/MeasureTheory/MeasurableSpace/Embedding.lean |
1 |
1 |
['github-actions'] |
nobody |
6-52101 6 days ago |
6-55722 6 days ago |
6-55767 6 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 |
6-48089 6 days ago |
39-3974 1 month ago |
39-4016 39 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 |
6-48006 6 days ago |
47-73894 1 month ago |
47-73937 47 days |
27437 |
kckennylau author:kckennylau |
feat(RingTheory/Valuation): some lemmas about comparing with 1 and 0 and with each other |
*From the 2025 Local Class Field Theory Workshop.*
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
109/22 |
Mathlib/NumberTheory/Padics/ValuativeRel.lean,Mathlib/RingTheory/Valuation/Basic.lean,Mathlib/RingTheory/Valuation/Extension.lean,Mathlib/RingTheory/Valuation/ValuativeRel.lean |
4 |
18 |
['erdOne', 'github-actions', 'kckennylau', 'matthewjasper', 'pechersky'] |
nobody |
6-46428 6 days ago |
8-58752 8 days ago |
8-58794 8 days |
27361 |
101damnations author:101damnations |
feat(Algebra/Homology/AlternatingConst): generalize to any appropriate complex shape and pair of maps |
Given an object `X : C` and endomorphisms `φ, ψ : X ⟶ X` such that `φ ∘ ψ = ψ ∘ φ = 0`, this PR defines the periodic chain and cochain complexes `... ⟶ X --φ--> X --ψ--> X --φ--> X --ψ--> 0` and `0 ⟶ X --ψ--> X --φ--> X --ψ--> X --φ--> ...` (or more generally for any complex shape `c` on `ℕ` where `c.Rel i j` implies `i` and `j` have different parity).
We calculate the homology of these periodic complexes.
This generalizes some of the current content of the file, which works for the chain complex where `ψ = 0` and `φ = Id`.
---
[](https://gitpod.io/from-referrer/)
|
maintainer-merge
t-algebra
label:t-algebra$ |
129/13 |
Mathlib/Algebra/Homology/AlternatingConst.lean |
1 |
3 |
['github-actions', 'kbuzzard'] |
nobody |
6-42268 6 days ago |
6-42268 6 days ago |
10-38782 10 days |
27527 |
peabrainiac author:peabrainiac |
feat(Topology): some `IsOpenMap` lemmas |
Some lemmas for `IsOpenMap` that I needed. I've also added variants for `IsClosedMap` to maintain symmetry in the API.
---
[](https://gitpod.io/from-referrer/)
|
t-topology |
46/0 |
Mathlib/Topology/Constructions.lean |
1 |
2 |
['github-actions', 'peabrainiac'] |
nobody |
6-30531 6 days ago |
6-31069 6 days ago |
6-31092 6 days |
26478 |
JovanGerb author:JovanGerb |
chore(LibraryRewrite): replace `rw??` with `rw?` |
As suggested by @YaelDillies, now `rw?` overwrites Lean core's implementation of `rw?`.
---
[](https://gitpod.io/from-referrer/)
|
t-meta |
56/49 |
Mathlib/Tactic/Widget/LibraryRewrite.lean,MathlibTest/LibraryRewrite.lean,MathlibTest/rewrites.lean |
3 |
5 |
['YaelDillies', 'erdOne', 'github-actions', 'leanprover-community-bot-assistant'] |
nobody |
6-25756 6 days ago |
6-36134 6 days ago |
21-11481 21 days |
27500 |
Komyyy author:Komyyy |
feat: the Riemann zeta function is meromorphic |
Also proves that the Hurwitz zeta function is meromorphic. This PR is split from #27499 to leave a good git diff history.
---
The `large-import` change occurs only in the new module, so it poses no problem.
- [x] depends on: #27499
This PR continues the work from #25597.
Original PR: https://github.com/leanprover-community/mathlib4/pull/25597 |
large-import
t-analysis
|
51/3 |
Mathlib.lean,Mathlib/Analysis/Meromorphic/Complex.lean,Mathlib/Analysis/Meromorphic/Gamma.lean |
3 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
6-19074 6 days ago |
6-19890 6 days ago |
6-20506 6 days |
27536 |
joelriou author:joelriou |
feat(Algebra/Homology): complementary embeddings |
Given two embeddings `e₁ : c₁.Embedding c` and `e₂ : c₂.Embedding c` of complex shapes, we introduce a property `e₁.AreComplementary e₂` saying that the image subsets of the indices of `c₁` and `c₂` form a partition of the indices of `c`.
If `e₁.IsTruncLE` and `e₂.IsTruncGE`, and `K : HomologicalComplex C c`, we construct a quasi-isomorphism `shortComplexTruncLEX₃ToTruncGE` between the cokernel of `K.ιTruncLE e₁ : K.truncLE e₁ ⟶ K` and `K.truncGE e₂`.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-category-theory
label:t-algebra$ |
327/0 |
Mathlib.lean,Mathlib/Algebra/Homology/Embedding/AreComplementary.lean |
2 |
1 |
['github-actions'] |
nobody |
5-82026 5 days ago |
5-82032 5 days ago |
5-82078 5 days |
27504 |
joelriou author:joelriou |
feat(CategoryTheory/Limits): filtered colimits of types |
In this file, given a functor `F : J ⥤ Type w₀` from a filtered category `J`, we compute the equivalence relation generated by `F.ColimitTypeRel` on `(j : J) × (F.obj j)`. Given `c : CoconeTypes F`, we deduce a lemma `Functor.CoconeTypes.injective_descColimitType_iff_of_isFiltered` which gives a concrete condition under which the map `F.descColimitType c : F.ColimitType → c.pt` is injective, which is an important step when proving `c.IsColimit`.
---
[](https://gitpod.io/from-referrer/)
|
t-category-theory |
134/0 |
Mathlib.lean,Mathlib/CategoryTheory/Limits/Types/ColimitType.lean,Mathlib/CategoryTheory/Limits/Types/ColimitTypeFiltered.lean |
3 |
5 |
['Ruben-VandeVelde', 'github-actions', 'joelriou'] |
nobody |
5-80291 5 days ago |
6-3435 6 days ago |
6-10289 6 days |
27537 |
vasnesterov author:vasnesterov |
feat(Analysis): radius of convergence for binomial series |
Introduce the binomial series as `FormalMultilinearSeries`, and prove that its radius of convergence is `1`.
---
- [x] depends on: #22518
[](https://gitpod.io/from-referrer/)
This PR continues the work from #22538.
Original PR: https://github.com/leanprover-community/mathlib4/pull/22538 |
t-analysis |
83/0 |
Mathlib.lean,Mathlib/Analysis/Analytic/Binomial.lean,Mathlib/RingTheory/Binomial.lean |
3 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
5-75649 5 days ago |
5-77046 5 days ago |
5-77098 5 days |
26270 |
vasnesterov author:vasnesterov |
chore(Analysis/Analytic): split `Analytic.Basic` |
Move the results on the radius of convergence from `Analytic/Basic.lean` to a new file `Analytic/ConvergenceRadius.lean`.
---
- [x] depends on: #26255
[](https://gitpod.io/from-referrer/)
|
tech debt
t-analysis
|
450/431 |
Mathlib.lean,Mathlib/Analysis/Analytic/Basic.lean,Mathlib/Analysis/Analytic/ConvergenceRadius.lean,Mathlib/Analysis/Analytic/OfScalars.lean,Mathlib/Analysis/Analytic/RadiusLiminf.lean |
5 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
5-75404 5 days ago |
5-75404 5 days ago |
6-65144 6 days |
27482 |
alreadydone author:alreadydone |
chore(RingTheory/SimpleModule): golf and generalize lifting_property |
---
Build succeeded but there's a strange post-build step error.
https://github.com/leanprover-community/mathlib4/actions/runs/16527173966/job/46744293147?pr=27482
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
11/14 |
Mathlib/RingTheory/SimpleModule/Basic.lean,Mathlib/RingTheory/SimpleModule/InjectiveProjective.lean |
2 |
2 |
['github-actions', 'smorel394'] |
nobody |
5-74231 5 days ago |
7-58041 7 days ago |
7-58026 7 days |
27548 |
euprunin author:euprunin |
chore(Control/Functor/Multivariate): remove use of `erw` in `f` (`private def f`) |
|
t-data |
1/1 |
Mathlib/Control/Functor/Multivariate.lean |
1 |
1 |
['github-actions'] |
nobody |
5-63100 5 days ago |
5-63106 5 days ago |
5-63158 5 days |
27550 |
chrisflav author:chrisflav |
chore(RingTheory/Polynomial): add `ker_constantCoeff` and `constantCoeff_surjective` |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
9/0 |
Mathlib/Algebra/Polynomial/Coeff.lean,Mathlib/RingTheory/Polynomial/Ideal.lean |
2 |
1 |
['github-actions'] |
nobody |
5-61901 5 days ago |
5-61972 5 days ago |
5-61956 5 days |
26798 |
robin-carlier author:robin-carlier |
feat(CategoryTheory/Monoidal/DayConvolution): `LawfulDayConvolutionMonoidalCategoryStruct` |
Given monoidal categories `C`, `V` and a category `D` with a pre-existing `MonoidalCategoryStruct`, we introduce a typeclass `LawfulDayConvolutionMonoidalCategoryStruct C V D` that bundles the required data and equations that the structure on `D` must have to be a monoidal subcategory of `C ⥤ V` if the latter was endowed with the day convolution monoidal structure.
The data in question is that of a faithful functor `ι : D ⥤ C ⥤ V`, as well as explicit natural transformations `ι.obj d ⊠ (ι.obj d') ⟶ tensor C ⋙ ι.obj (d ⊗ d')` that exhibit `ι.obj (d ⊗ d')` as a Day convolution of `ι.obj d` and `(ι.obj d')`, as well as similar data asserting that `ι.obj (𝟙_ D)` is a Day convolution unit. The equations required are identical to the ones that characterize the unitors and associators for Day convolution with respect to the Kan extensions units.
Given such a structure, using that the corresponding relations hold in `C ⥤ V`, we show that the monoidal category structure on `D` defines a `MonoidalCategory D`, i.e that all the required equations such as the pentagon/triangular equalities, bifunctoriality of the tensor product etc. are satisfied. Thus, we can think of `LawfulDayConvolutionMonoidalCategoryStruct C V D` as a constructor for monoidal categories.
While this is a step towards a Day convolution monoidal structure in (a type alias) `C ⥤ V`, the framework is yet incomplete, as it assumes a pre-existing monoidal category structure. We will give constructors for (`MonoidalCategoryStruct` and) `LawfulDayConvolutionMonoidalCategoryStruct C V D` with various degree of definitional control over the resulting structure in a forthcoming PR.
---
- [x] depends on: #25757
I recommend the reviewer to at least have a glance at #26820 to see where this is going, and how this one fits in the design I have in mind.
[](https://gitpod.io/from-referrer/)
|
t-category-theory |
336/8 |
Mathlib/CategoryTheory/Monoidal/DayConvolution.lean |
1 |
4 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
5-61382 5 days ago |
5-61405 5 days ago |
19-37483 19 days |
27554 |
euprunin author:euprunin |
chore(LinearAlgebra/PiTensorProduct): `grind` away use of `erw` in `lifts_zero` |
|
t-algebra label:t-algebra$ |
1/1 |
Mathlib/LinearAlgebra/PiTensorProduct.lean |
1 |
1 |
['github-actions'] |
nobody |
5-56538 5 days ago |
5-56549 5 days ago |
5-56594 5 days |
26031 |
joelriou author:joelriou |
feat(Algebra/Homology): the derived category of a linear abelian category is linear |
---
- [x] depends on: #25931
This PR continues the work from #24596.
Original PR: https://github.com/leanprover-community/mathlib4/pull/24596 |
t-category-theory |
71/0 |
Mathlib.lean,Mathlib/Algebra/Homology/DerivedCategory/Linear.lean,Mathlib/Algebra/Homology/HomotopyCategory/Shift.lean,Mathlib/Algebra/Homology/HomotopyCategory/SingleFunctors.lean |
4 |
n/a |
['AntoineChambert-Loir', 'github-actions', 'joelriou', 'mathlib4-dependent-issues-bot'] |
nobody |
5-49143 5 days ago |
unknown |
unknown |
27566 |
wwylele author:wwylele |
feat(Data/Real): Archimedean.embedReal is a ring hom when M is an ordered ring |
Also shows that this ends up the same as `LinearOrderedField.inducedOrderRingHom` for fields
---
This is a spin-off from #27268 ~~because I got bored~~ . This is not in a high priority as I don't need it for anything yet, but the last lemma shows that `embedReal` is a generalization of `LinearOrderedField.inducedOrderRingHom` (which is only stated for field, and I didn't find when I was making the group embedding). Perhaps we should refactor `Mathlib/Algebra/Order/CompleteField.lean` with the definition here. Indeed, if we replace every `ℝ` with `(R : Type*)[ConditionallyCompleteLinearOrderedField R]` in `Data/Real/Embedding.lean`, the proof still works. What do you think?
[](https://gitpod.io/from-referrer/)
|
large-import
t-data
|
220/3 |
Mathlib/Data/Real/Embedding.lean |
1 |
1 |
['github-actions'] |
nobody |
5-43071 5 days ago |
5-43078 5 days ago |
5-43131 5 days |
27567 |
themathqueen author:themathqueen |
feat(LinearAlgebra/TensorProduct/Tower): add `lid` and `assoc` tensor lemmas |
This adds `TensorProduct.lid_tensor` and `TensorProduct.assoc_tensor`.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
21/0 |
Mathlib/LinearAlgebra/TensorProduct/Tower.lean |
1 |
2 |
['github-actions', 'themathqueen'] |
nobody |
5-41567 5 days ago |
5-42359 5 days ago |
5-42404 5 days |
27288 |
themathqueen author:themathqueen |
feat(LinearAlgebra/TensorProduct/Basic): semi-linearize `map` and `lift` |
Semi-linearizing `TensorProduct.map`. Part of #27353.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
29/18 |
Mathlib/Algebra/Category/ModuleCat/ChangeOfRings.lean,Mathlib/LinearAlgebra/TensorProduct/Basic.lean,Mathlib/RingTheory/Coalgebra/Hom.lean |
3 |
4 |
['ADedecker', 'eric-wieser', 'github-actions', 'themathqueen'] |
nobody |
5-40367 5 days ago |
5-40367 5 days ago |
8-64892 8 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 |
22 |
['alreadydone', 'erdOne', 'eric-wieser', 'github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'leanprover-community-mathlib4-bot', 'mathlib4-dependent-issues-bot'] |
erdOne assignee:erdOne |
5-35224 5 days ago |
5-45014 5 days ago |
108-35052 108 days |
27544 |
eric-wieser author:eric-wieser |
feat: upgrade lflip to a `LinearEquiv` |
This deletes some `aux` definitions without deprecation.
This is helpful for building the version of `DFinsupp.lsum` for bilinear maps.
A handful of existing users of `lflip` now need to add an explicit `toLinearMap`.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
24/35 |
Mathlib/LinearAlgebra/BilinearForm/Basic.lean,Mathlib/LinearAlgebra/BilinearMap.lean,Mathlib/LinearAlgebra/TensorPower/Basic.lean,Mathlib/LinearAlgebra/TensorProduct/Associator.lean,Mathlib/LinearAlgebra/TensorProduct/Graded/External.lean,Mathlib/LinearAlgebra/TensorProduct/Tower.lean,Mathlib/RingTheory/PiTensorProduct.lean,Mathlib/RingTheory/TensorProduct/Basic.lean |
8 |
1 |
['github-actions'] |
nobody |
5-34754 5 days ago |
5-34754 5 days ago |
5-35097 5 days |
27562 |
hrmacbeth author:hrmacbeth |
chore: deduplicate "transform at location" methods |
Many metaprograms have the following general structure: the input is an expression `e` and the output is a new expression `e'`, together with a proof that `e = e'`. Such a metaprogram produces a variety of tactics: it may be used to modify the goal, a specified hypothesis, or (via `Tactic.Location`) a combination of these.
Roughly the same code for this is repeated throughout the library, for the tactics `ring_nf`, `abel_nf`, `norm_num`, `push_neg` and `reduce_mod_char`; possibly it originates from the `ring_nf` version, #552.
This PR extracts this repeated code to a stand-alone function in `Mathlib.Util.AtLocation`.
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-meta
|
115/166 |
Mathlib.lean,Mathlib/Tactic/Abel.lean,Mathlib/Tactic/NormNum/Core.lean,Mathlib/Tactic/Push.lean,Mathlib/Tactic/ReduceModChar.lean,Mathlib/Tactic/Ring/RingNF.lean,Mathlib/Util/AtLocation.lean,MathlibTest/abel.lean,MathlibTest/norm_num.lean |
9 |
4 |
['github-actions', 'grunweg', 'hrmacbeth'] |
nobody |
5-28401 5 days ago |
5-28401 5 days ago |
5-48410 5 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 |
3 |
['YaelDillies', 'github-actions', 'leanprover-community-bot-assistant'] |
nobody |
5-26713 5 days ago |
5-26737 5 days ago |
50-75419 50 days |
27018 |
Komyyy author:Komyyy |
feat: Finite product of Alexandrov-discrete spaces is Alexandrov-discrete |
---
- [x] depends on: #27016
[](https://gitpod.io/from-referrer/)
|
t-topology |
93/9 |
Mathlib/Data/Set/Lattice.lean,Mathlib/Data/Set/Lattice/Image.lean,Mathlib/Order/Filter/Ker.lean,Mathlib/Topology/AlexandrovDiscrete.lean,Mathlib/Topology/NhdsKer.lean |
5 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
5-5460 5 days ago |
5-18447 5 days ago |
5-18431 5 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 |
14/0 |
Mathlib/AlgebraicGeometry/Properties.lean,Mathlib/AlgebraicGeometry/Scheme.lean |
2 |
4 |
['Raph-DG', 'github-actions', 'joelriou', 'leanprover-community-bot-assistant'] |
nobody |
5-5255 5 days ago |
5-5255 5 days ago |
40-71303 40 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 |
5-2479 5 days ago |
66-64559 2 months ago |
72-68952 72 days |
27283 |
Louddy author:Louddy |
feat(SkewMonoidAlgebra): 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 |
5-2340 5 days ago |
14-4926 14 days ago |
14-4976 14 days |
27253 |
Louddy author:Louddy |
feat(SkewMonoidAlgebra): 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 |
5-2318 5 days ago |
14-67254 14 days ago |
14-67267 14 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
|
94/35 |
Mathlib/Analysis/Convex/Cone/Basic.lean,Mathlib/Geometry/Convex/Cone/Basic.lean |
2 |
8 |
['YaelDillies', 'b-mehta', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
4-86017 4 days ago |
5-79929 5 days ago |
43-31856 43 days |
27582 |
IvanRenison author:IvanRenison |
feat(Combinatorics/SimpleGraph/Paths): add theorem `SimpleGraph.Walk.IsPath.isPath_concat` |
This contribution was created as part of the Utrecht Summerschool "Formalizing Mathematics in Lean" in July 2025.
---
[](https://gitpod.io/from-referrer/)
|
t-combinatorics |
7/0 |
Mathlib/Combinatorics/SimpleGraph/Paths.lean |
1 |
1 |
['github-actions'] |
nobody |
4-84798 4 days ago |
4-84824 4 days ago |
4-84874 4 days |
27583 |
RemyDegenne author:RemyDegenne |
feat: in a countable discrete measurable space, every measure is s-finite |
The instance is placed in the `WithDensity` file, because that's where we have the instance `SFinite (c • μ)` that I use in the proof.
---
[](https://gitpod.io/from-referrer/)
|
t-measure-probability |
4/0 |
Mathlib/MeasureTheory/Measure/WithDensity.lean |
1 |
1 |
['github-actions'] |
nobody |
4-84759 4 days ago |
4-84762 4 days ago |
4-84809 4 days |
27581 |
eric-wieser author:eric-wieser |
fix(Data/BitVec): remove a `SMul` instance diamond |
When the `Nat`- and `Int`-action typeclasses and their instances were upstreamed, they changed to a different (and worse) defeq.
This removes the mathlib instances and proves the old defeq still holds propositionally.
Also move some theorems out of the `BitVec` file that are not about `BitVec` at all, and are about `Fin`.
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-data
|
57/54 |
Mathlib/Data/BitVec.lean,Mathlib/Data/ZMod/Defs.lean |
2 |
2 |
['eric-wieser', 'github-actions'] |
nobody |
4-84289 4 days ago |
5-175 5 days ago |
5-227 5 days |
27584 |
RemyDegenne author:RemyDegenne |
feat(Probability): lemmas about `Kernel.discard` |
---
[](https://gitpod.io/from-referrer/)
|
t-measure-probability |
22/1 |
Mathlib/MeasureTheory/Measure/GiryMonad.lean,Mathlib/Probability/Kernel/Basic.lean,Mathlib/Probability/Kernel/Composition/Comp.lean,Mathlib/Probability/Kernel/Composition/MeasureComp.lean |
4 |
1 |
['github-actions'] |
nobody |
4-82998 4 days ago |
4-83005 4 days ago |
4-83054 4 days |
27585 |
RemyDegenne author:RemyDegenne |
feat(Probability): `posterior_eq_withDensity_of_countable` |
This PR adds a simpler version of `posterior_eq_withDensity` for the case of a countable space.
---
[](https://gitpod.io/from-referrer/)
|
t-measure-probability |
12/0 |
Mathlib/Probability/Kernel/Posterior.lean |
1 |
1 |
['github-actions'] |
nobody |
4-82739 4 days ago |
4-82751 4 days ago |
4-82797 4 days |
27586 |
RemyDegenne author:RemyDegenne |
feat(Probability): `Kernel.comp_const` |
`κ ∘ₖ Kernel.const α μ = Kernel.const α (κ ∘ₘ μ)`
---
[](https://gitpod.io/from-referrer/)
|
t-measure-probability |
7/0 |
Mathlib/Probability/Kernel/Composition/MeasureComp.lean |
1 |
1 |
['github-actions'] |
nobody |
4-82450 4 days ago |
4-82462 4 days ago |
4-82508 4 days |
26016 |
CBirkbeck author:CBirkbeck |
Iterated derivatives of tsum's within some open set. |
We add some IteratedDerivWithin versions of deriv_tsum using the new SummableLocallyUniformly API.
This PR continues the work from #25096.
Original PR: https://github.com/leanprover-community/mathlib4/pull/25096 |
t-analysis |
139/0 |
Mathlib.lean,Mathlib/Algebra/BigOperators/Pi.lean,Mathlib/Analysis/Calculus/IteratedDeriv/Lemmas.lean,Mathlib/Topology/Algebra/InfiniteSum/TsumUniformlyOn.lean,Mathlib/Topology/Algebra/InfiniteSum/UniformOn.lean |
5 |
3 |
['CBirkbeck', 'github-actions', 'leanprover-community-bot-assistant'] |
nobody |
4-82377 4 days ago |
4-86104 4 days ago |
27-40018 27 days |
27587 |
RemyDegenne author:RemyDegenne |
feat(Probability): instances for `Kernel` on empty types |
---
[](https://gitpod.io/from-referrer/)
|
t-measure-probability |
20/0 |
Mathlib/Probability/Kernel/Basic.lean,Mathlib/Probability/Kernel/Defs.lean |
2 |
1 |
['github-actions'] |
nobody |
4-80086 4 days ago |
4-80092 4 days ago |
4-80140 4 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
|
859/5 |
Mathlib/Combinatorics/Additive/VerySmallDoubling.lean |
1 |
61 |
['YaelDillies', 'github-actions', 'strihanje01'] |
nobody |
4-60842 4 days ago |
21-49914 21 days ago |
27-13734 27 days |
27597 |
mitchell-horner author:mitchell-horner |
feat(Combinatorics/SimpleGraph): define `completeEquipartiteGraph` |
Define the complete equipartite graph in `r` parts each of *equal* size `t` such that two vertices are adjacent if and only if they are in different parts.
These graphs are typically denoted by $$K_r(t)$$.
---
I'm not 100% certain these definitions need their own file. I've placed them at the bottom of `CompleteMultipartite.lean` as complete equipartite graphs are just a special case of complete multipartite graphs.
However, I intend to PR another definition `completeEquipartiteSubgraph`. In which case it might be appropriate to create a new file `CompleteEquipartite.lean` that contains both definitions.
[](https://gitpod.io/from-referrer/)
|
large-import
t-combinatorics
|
128/0 |
Mathlib/Combinatorics/SimpleGraph/Coloring.lean,Mathlib/Combinatorics/SimpleGraph/CompleteMultipartite.lean |
2 |
1 |
['github-actions'] |
nobody |
4-60280 4 days ago |
4-61026 4 days ago |
4-61090 4 days |
27600 |
ocfnash author:ocfnash |
feat: miscellaneous Lie algebra lemmas |
These came up in the proof that the Geck Construction yields _semisimple_ Lie algebras. I am splitting them into their own PR to simplify review.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
86/14 |
Mathlib/Algebra/Lie/Abelian.lean,Mathlib/Algebra/Lie/Basic.lean,Mathlib/Algebra/Lie/Semisimple/Defs.lean,Mathlib/Algebra/Lie/Subalgebra.lean |
4 |
1 |
['github-actions'] |
nobody |
4-53115 4 days ago |
4-56987 4 days ago |
4-56971 4 days |
27602 |
mitchell-horner author:mitchell-horner |
feat(Combinatorics/SimpleGraph): define `completeBipartiteSubgraph` |
Define the complete bipartite subgraphs of `s` and `t` parts as a "left" subset of `s` vertices and a "right" subset of `t` vertices such that every vertex in the "left" subset is adjacent to every vertex in the "right" subset.
In this case `Nonempty (G.completeBipartiteSubgraph (card α) (card β))` is equivalent to `completeBipartiteGraph α β ⊑ G`, that is, finding a "left" subset of `s` vertices and a "right" subset of `t` vertices such that every vertex in the "left" subset is adjacent to every vertex in the "right" subset is equivalent to finding an injective homomorphism `completeBipartiteGraph α β` to `G`.
---
[](https://gitpod.io/from-referrer/)
|
t-combinatorics |
88/0 |
Mathlib/Combinatorics/SimpleGraph/Bipartite.lean |
1 |
1 |
['github-actions'] |
nobody |
4-52344 4 days ago |
4-53979 4 days ago |
4-54030 4 days |
27467 |
themathqueen author:themathqueen |
chore(LinearAlgebra/BilinearMap): semi-linearize |
Semi-linearizes `llcomp` and creates a new definition `compr₂ₛₗ` for the semi-linear version of `compr₂`.
Original PRs: #27353 (#27310, #24208).
Co-authored-by: @ADedecker
---
[](https://gitpod.io/from-referrer/)
|
maintainer-merge
t-algebra
label:t-algebra$ |
78/30 |
Mathlib/Algebra/Module/Equiv/Defs.lean,Mathlib/LinearAlgebra/BilinearMap.lean |
2 |
16 |
['eric-wieser', 'github-actions', 'j-loreaux', 'themathqueen'] |
nobody |
4-41215 4 days ago |
4-41215 4 days ago |
6-60628 6 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 |
8 |
['Komyyy', 'digama0', 'eric-wieser', 'github-actions'] |
nobody |
4-27616 4 days ago |
19-62001 19 days ago |
19-61986 19 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 |
16 |
['YaelDillies', 'eric-wieser', 'github-actions', 'j-loreaux', 'leanprover-community-bot-assistant', 'mathlib-bors'] |
nobody |
4-15771 4 days ago |
79-69822 2 months ago |
164-42855 164 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
|
78/0 |
Mathlib/MeasureTheory/Measure/Restrict.lean |
1 |
3 |
['RemyDegenne', 'github-actions', 'js2357'] |
nobody |
4-14884 4 days ago |
4-14884 4 days ago |
12-39595 12 days |
27385 |
grunweg author:grunweg |
feat: weaken definiteness requirement for `ENormed(Add)(Comm)Monoid`s |
Most lemmas about these do not require the enorm to be positive definite (i.e., work fine if a nontrivial element has zero enorm), or can be rephrased easily. A handful of lemmas do require this condition.
Weaken the definition of `ENormed(Add)(Comm)Monoid`s to only ask that zero have enorm zero, and
add new classes `StrictENormed(Add)(Comm)Monoid` which also ask for definiteness.
Most existing lemmas are kept unchanged (i.e., have slightly weaker hypotheses now);
a few have their typeclasses adjusted.
The motivating example behind this is `eLpNorm`, which is an enormed commutative (additive) monoid --- when we drop the definiteness requirement. This will (hopefully) allow unifying many lemma about `eLpNorm` with their more general enorm variants.
---
[](https://gitpod.io/from-referrer/)
|
carleson
t-analysis
|
94/39 |
Mathlib/Analysis/Normed/Group/Basic.lean,Mathlib/Analysis/Normed/Group/Continuity.lean,Mathlib/Analysis/NormedSpace/PiTensorProduct/InjectiveSeminorm.lean,Mathlib/MeasureTheory/Function/LpSeminorm/Basic.lean,Mathlib/MeasureTheory/Integral/IntegrableOn.lean,Mathlib/MeasureTheory/Integral/IntervalIntegral/Basic.lean |
6 |
5 |
['github-actions', 'grunweg', 'sgouezel'] |
nobody |
4-3890 4 days ago |
8-48872 8 days ago |
8-48857 8 days |
27633 |
Ruben-VandeVelde author:Ruben-VandeVelde |
feat: MvPolynomial.coeff_mapRange |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
5/5 |
Mathlib/Algebra/MvPolynomial/Basic.lean,Mathlib/Algebra/MvPolynomial/Eval.lean |
2 |
1 |
['github-actions'] |
nobody |
3-78577 3 days ago |
3-78581 3 days ago |
3-78631 3 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
|
103/0 |
Mathlib/Data/Sum/Basic.lean,Mathlib/Topology/Constructions/SumProd.lean |
2 |
6 |
['ADedecker', 'github-actions', 'grunweg'] |
nobody |
3-74369 3 days ago |
44-65543 1 month ago |
44-65534 44 days |
27605 |
ocfnash author:ocfnash |
feat: basic linear algebra lemmas about matrices |
These came up in the proof that the Geck Construction yields semisimple Lie algebras. I am splitting them into their own PR to simplify review.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
112/6 |
Mathlib/Analysis/Normed/Module/FiniteDimension.lean,Mathlib/Data/Matrix/Block.lean,Mathlib/Data/Matrix/Diagonal.lean,Mathlib/Data/Matrix/Mul.lean,Mathlib/LinearAlgebra/Basis/Basic.lean,Mathlib/LinearAlgebra/Basis/Defs.lean,Mathlib/LinearAlgebra/Eigenspace/Basic.lean,Mathlib/LinearAlgebra/Eigenspace/Matrix.lean,Mathlib/LinearAlgebra/Matrix/BilinearForm.lean,Mathlib/LinearAlgebra/Matrix/ToLin.lean,Mathlib/LinearAlgebra/Pi.lean |
11 |
9 |
['github-actions', 'j-loreaux', 'ocfnash', 'themathqueen'] |
nobody |
3-73268 3 days ago |
3-73268 3 days ago |
4-4983 4 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/)
|
new-contributor
t-dynamics
|
34/0 |
Mathlib.lean,Mathlib/Dynamics/MeasurePreserving/Lemmas.lean |
2 |
1 |
['github-actions'] |
nobody |
3-72028 3 days ago |
3-72092 3 days ago |
21-55392 21 days |
27471 |
FrankieNC author:FrankieNC |
feat(Topology/Baire/Lemmas): In a nonempty Baire space, any dense GDelta set is not meagre |
Proves that in a nonempty Baire space any dense Gδ set is not meagre
---
[](https://gitpod.io/from-referrer/)
|
t-topology |
7/0 |
Mathlib/Topology/Baire/Lemmas.lean |
1 |
2 |
['FrankieNC', 'github-actions'] |
nobody |
3-70074 3 days ago |
7-67404 7 days ago |
7-67456 7 days |
27635 |
Ruben-VandeVelde author:Ruben-VandeVelde |
chore: deprecate SubsemiringClass.coe_pow |
---
[](https://gitpod.io/from-referrer/)
|
|
2/7 |
Mathlib/Algebra/Ring/Subsemiring/Defs.lean,Mathlib/Analysis/Normed/Ring/Basic.lean |
2 |
3 |
['Ruben-VandeVelde', 'github-actions', 'grunweg'] |
nobody |
3-69593 3 days ago |
3-69593 3 days ago |
3-72592 3 days |
27320 |
Jlh18 author:Jlh18 |
doc (CategoryTheory/Bicategory/Grothendieck): rename Grothendieck to coGrothendieck |
Rename `CategoryTheory.Pseudofunctor.Grothendieck` to `CategoryTheory.Pseudofunctor.coGrothendieck`. Currently there are two inconsistent conventions taken in [`CategoryTheory.Grothendieck`](https://leanprover-community.github.io/mathlib4_docs/Mathlib/CategoryTheory/Grothendieck.html#CategoryTheory.Grothendieck) and [`CategoryTheory.Pseudofunctor.Grothendieck`](https://leanprover-community.github.io/mathlib4_docs/Mathlib/CategoryTheory/Bicategory/Grothendieck.html#CategoryTheory.Pseudofunctor.Grothendieck), namely the latter includes an `op` on the indexing category / base category of the Grothendieck construction.
Later on, I will make more PRs to introduce the version of `CategoryTheory.Pseudofunctor.Grothendieck` that does not have an `op`.
Zulip discussion: [#mathlib4 > Refactor Grothendieck from Pseudofunctor.Grothendieck](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Refactor.20Grothendieck.20from.20Pseudofunctor.2EGrothendieck/with/529165679).
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-category-theory
|
46/38 |
Mathlib/CategoryTheory/Bicategory/Grothendieck.lean,Mathlib/CategoryTheory/FiberedCategory/Grothendieck.lean |
2 |
5 |
['Jlh18', 'github-actions', 'joelriou', 'kckennylau'] |
nobody |
3-68597 3 days ago |
3-68747 3 days ago |
9-83790 9 days |
27636 |
Louddy author:Louddy |
feat(Bivariate): aevalAeval and swap |
Add the `aeval` equivalent to `Bivariate.evalEval`.
This PR also introduces `Bivariate.swap`, the R-algebra automorphism given by `X ↦ Y` and `Y ↦ X`.
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$ |
45/0 |
Mathlib/Algebra/Polynomial/Bivariate.lean |
1 |
1 |
['github-actions'] |
nobody |
3-66865 3 days ago |
3-66912 3 days ago |
3-66921 3 days |
26842 |
oliver-butterley author:oliver-butterley |
feat(Mathlib/Dynamics/BirkhoffSum/Average): add lemma `birkhoffAverage_of_invariant` |
If a function `g` is invariant under a function `f` (i.e., `g ∘ f = g`), then the Birkhoff average of `g` over `f` for `n` iterations is equal to `g`. Requires that `0 < n`.
Co-authored-by: Lua Viana Reis
- [x] depends on: #26810
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
easy
|
10/0 |
Mathlib/Dynamics/BirkhoffSum/Average.lean |
1 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
3-66200 3 days ago |
3-66223 3 days ago |
3-67111 3 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', 'madvorak'] |
nobody |
3-65660 3 days ago |
21-47284 21 days ago |
21-57309 21 days |
27639 |
staroperator author:staroperator |
feat(Algebra/Order/Sub): `Sub` instance for linearly canonically ordered monoid |
There is a `Sub` instance for linearly canonically ordered monoid using choice that satisfies `OrderedSub`.
---
Thanks @eric-wieser for the suggestion in #27341!
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
28/0 |
Mathlib/Algebra/Order/Sub/Basic.lean |
1 |
1 |
['github-actions'] |
nobody |
3-65117 3 days ago |
3-65128 3 days ago |
3-65175 3 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 |
t-topology |
24/9 |
Mathlib/Topology/Separation/Hausdorff.lean,Mathlib/Topology/Sober.lean |
2 |
20 |
['faenuccio', 'github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'plp127'] |
nobody |
3-63124 3 days ago |
3-67631 3 days ago |
38-67823 38 days |
27598 |
ocfnash author:ocfnash |
feat: a finite union of proper submodules is a proper subset |
(provided the coefficients are a sufficiently large field).
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
135/1 |
Mathlib.lean,Mathlib/Algebra/Module/Submodule/Union.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/Data/Finset/Card.lean,Mathlib/Data/Set/Card.lean |
5 |
1 |
['github-actions'] |
nobody |
3-62344 3 days ago |
4-58733 4 days ago |
4-58717 4 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 |
130/121 |
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 |
6 |
['Parcly-Taxel', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'madvorak'] |
nobody |
3-61316 3 days ago |
3-61335 3 days ago |
48-53827 48 days |
27333 |
FrankieNC author:FrankieNC |
feat: in a Baire space, every nonempty open set is of second category |
In a Baire space, every nonempty open set is non‑meagre (of second category).
---
[](https://gitpod.io/from-referrer/)
|
maintainer-merge
t-topology
|
10/0 |
Mathlib/Topology/Baire/Lemmas.lean |
1 |
13 |
['FrankieNC', 'b-mehta', 'github-actions', 'grunweg'] |
nobody |
3-59099 3 days ago |
3-69571 3 days ago |
11-36570 11 days |
27642 |
themathqueen author:themathqueen |
feat(Analysis/InnerProductSpace/Projection): define symmetric projections |
This pr defines symmetric projections (`LinearMap.IsSymmetricProjection`) which are simply symmetric idempotents. This generalizes most of the results concerning star projection operators (since it needs completeness). In a complete space, these two definitions obviously coincide.
An operator `p` is a symmetric projection if and only if it equals `(range p).starProjection`. This is a more general version of [isStarProjection_iff_eq_starProjection_range](https://leanprover-community.github.io/mathlib4_docs/Mathlib/Analysis/InnerProductSpace/Adjoint.html#isStarProjection_iff_eq_starProjection_range).
---
[](https://gitpod.io/from-referrer/)
|
t-analysis |
81/19 |
Mathlib/Analysis/InnerProductSpace/Adjoint.lean,Mathlib/Analysis/InnerProductSpace/Projection.lean,Mathlib/Analysis/InnerProductSpace/Symmetric.lean |
3 |
1 |
['github-actions'] |
nobody |
3-58678 3 days ago |
3-59343 3 days ago |
3-59397 3 days |
27638 |
plp127 author:plp127 |
feat: subsingleton `ℕ` and `ℤ` modules |
Provide some instances `AddCommMonoid.subsingletonNatModule` and `AddCommMonoid.subsingletonIntModule`. Also move some of the theorems about `ℕ` and `ℤ` modules from `Algebra/Module/End` to `Algebra/Module/NatInt`.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
53/45 |
Mathlib/Algebra/Algebra/Rat.lean,Mathlib/Algebra/Module/End.lean,Mathlib/Algebra/Module/NatInt.lean,Mathlib/Algebra/Module/Submodule/RestrictScalars.lean,Mathlib/Data/ZMod/Basic.lean,Mathlib/RingTheory/OreLocalization/Ring.lean |
6 |
3 |
['github-actions', 'plp127'] |
nobody |
3-58389 3 days ago |
3-65591 3 days ago |
3-65637 3 days |
27634 |
agjftucker author:agjftucker |
fix(Analysis/Calculus/Implicit): consistently rename {`map`, `fun`, `function`} to `fun` |
There are several clear naming issues in the file Implicit.lean, such as
```
theorem prod_map_implicitFunction :
∀ᶠ p : F × G in 𝓝 (φ.prodFun φ.pt), φ.prodFun (φ.implicitFunction p.1 p.2) = p :=
```
where `prod_map` and `prodFun` both refer to the same thing. In this PR I have done my best to resolve these as consistently as possible by renaming everything `map`, also everything `function`, to `fun`. This has the added benefit of making some long names a little shorter.
In passing I rewrapped some comments and replaced `haveI` with `have` where it had been used like `haveI` in Lean 3.
Moves:
- ImplicitFunctionData -> ImplicitFunData
- ImplicitFunctionData.implicitFunction -> ImplicitFunData.implicitFun
- ImplicitFunctionData.prod_map_implicitFunction -> ImplicitFunData.prodFun_implicitFun
- ImplicitFunctionData.left_map_implicitFunction -> ImplicitFunData.leftFun_implicitFun
- ImplicitFunctionData.right_map_implicitFunction -> ImplicitFunData.rightFun_implicitFun
- ImplicitFunctionData.implicitFunction_apply_image -> ImplicitFunData.implicitFun_apply_image
- ImplicitFunctionData.implicitFunction_hasStrictFDerivAt -> ImplicitFunData.hasStrictFDerivAt_implicitFun
- HasStrictFDerivAt.implicitFunctionDataOfComplemented -> HasStrictFDerivAt.implicitFunDataOfComplemented
- HasStrictFDerivAt.implicitFunctionOfComplemented -> HasStrictFDerivAt.implicitFunOfComplemented
- HasStrictFDerivAt.map_implicitFunctionOfComplemented_eq -> HasStrictFDerivAt.map_implicitFunOfComplemented_eq
- HasStrictFDerivAt.eq_implicitFunctionOfComplemented -> HasStrictFDerivAt.eq_implicitFunOfComplemented
- HasStrictFDerivAt.implicitFunctionOfComplemented_apply_image -> HasStrictFDerivAt.implicitFunOfComplemented_apply_image
- HasStrictFDerivAt.to_implicitFunctionOfComplemented -> HasStrictFDerivAt.to_implicitFunOfComplemented
- HasStrictFDerivAt.implicitFunction -> HasStrictFDerivAt.implicitFun
- HasStrictFDerivAt.tendsto_implicitFunction -> HasStrictFDerivAt.tendsto_implicitFun
- _root_.Filter.Tendsto.implicitFunction -> _root_.Filter.Tendsto.implicitFun
- HasStrictFDerivAt.map_implicitFunction_eq -> HasStrictFDerivAt.map_implicitFun_eq
- HasStrictFDerivAt.implicitFunction_apply_image -> HasStrictFDerivAt.implicitFun_apply_image
- HasStrictFDerivAt.eq_implicitFunction -> HasStrictFDerivAt.eq_implicitFun
- HasStrictFDerivAt.to_implicitFunction -> HasStrictFDerivAt.to_implicitFun
---
[](https://gitpod.io/from-referrer/)
|
t-analysis
easy
|
165/121 |
Mathlib/Analysis/Calculus/Implicit.lean,docs/1000.yaml,docs/overview.yaml,docs/undergrad.yaml |
4 |
1 |
['github-actions'] |
nobody |
3-53502 3 days ago |
3-74948 3 days ago |
3-74997 3 days |
27649 |
hrmacbeth author:hrmacbeth |
chore: deduplicate "recursively on atoms" code |
This PR abstracts the "run recursively on atoms" method, implicit in `ring_nf` and `atom_nf`, for stand-alone use. The key function produced is
```lean
def Mathlib.Tactic.AtomM.recurse
(s : IO.Ref AtomM.State)
(cfg : AtomM.Recurse.Config)
(eval : Expr → AtomM Simp.Result)
(cleanup : Simp.Result → MetaM Simp.Result)
(tgt : Expr) :
MetaM Simp.Result
```
which runs an input metaprogram `(eval : Expr → AtomM Simp.Result)` on an input expression `tgt` *recursively*: on each atom for the metaprogram `eval`, before packaging it as an atom, it finds the maximal subexpressions of that atom on which `eval` is applicable, and runs `eval` there too (and so on).
Also rewrite `ring_nf` and `atom_nf` to use the abstracted method.
---
[](https://gitpod.io/from-referrer/)
|
t-meta |
190/131 |
Mathlib.lean,Mathlib/Tactic/Abel.lean,Mathlib/Tactic/Ring/RingNF.lean,Mathlib/Util/AtomM/Recurse.lean,MathlibTest/ring.lean |
5 |
1 |
['github-actions'] |
nobody |
3-40397 3 days ago |
3-40412 3 days ago |
3-42580 3 days |
27655 |
euprunin author:euprunin |
chore(Geometry/RingedSpace): remove use of `erw` in `ofRestrict_top_c` |
|
t-algebraic-geometry |
1/3 |
Mathlib/Geometry/RingedSpace/PresheafedSpace.lean |
1 |
1 |
['github-actions'] |
nobody |
3-37243 3 days ago |
3-37246 3 days ago |
3-37293 3 days |
27656 |
euprunin author:euprunin |
chore(Geometry/RingedSpace): remove use of `erw` in `stalkSpecializes_stalkMap` |
|
t-algebraic-geometry |
1/2 |
Mathlib/Geometry/RingedSpace/Stalks.lean |
1 |
1 |
['github-actions'] |
nobody |
3-36905 3 days ago |
3-36918 3 days ago |
3-36963 3 days |
27657 |
euprunin author:euprunin |
chore(Geometry/RingedSpace): remove use of `erw` in `forget_preservesLimitsOfLeft` |
|
t-algebraic-geometry |
5/2 |
Mathlib/Geometry/RingedSpace/OpenImmersion.lean |
1 |
1 |
['github-actions'] |
nobody |
3-36560 3 days ago |
3-36572 3 days ago |
3-36619 3 days |
27658 |
euprunin author:euprunin |
chore(Geometry/RingedSpace): remove use of `erw` in `app_inv_app'` |
|
t-algebraic-geometry |
3/1 |
Mathlib/Geometry/RingedSpace/OpenImmersion.lean |
1 |
1 |
['github-actions'] |
nobody |
3-36248 3 days ago |
3-36253 3 days ago |
3-36299 3 days |
27659 |
euprunin author:euprunin |
chore(Geometry/RingedSpace): remove use of `erw` in `vPullbackConeIsLimit` |
|
t-algebraic-geometry |
4/1 |
Mathlib/Geometry/RingedSpace/PresheafedSpace/Gluing.lean |
1 |
1 |
['github-actions'] |
nobody |
3-35865 3 days ago |
3-35870 3 days ago |
3-35915 3 days |
27660 |
euprunin author:euprunin |
chore(Geometry/RingedSpace): remove use of `erw` in `isUnit_of_isUnit_germ` |
|
t-algebraic-geometry |
2/3 |
Mathlib/Geometry/RingedSpace/Basic.lean |
1 |
1 |
['github-actions'] |
nobody |
3-35636 3 days ago |
3-35662 3 days ago |
3-35711 3 days |
27665 |
pechersky author:pechersky |
chore(Algebra/Group/WithOne): With{One,Zero}.coe_injective |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
easy
label:t-algebra$ |
4/0 |
Mathlib/Algebra/Group/WithOne/Defs.lean |
1 |
1 |
['github-actions'] |
nobody |
3-14030 3 days ago |
3-14204 3 days ago |
3-14201 3 days |
26689 |
euprunin author:euprunin |
chore: golf Combinatorics/ using `grind` |
|
t-combinatorics |
9/62 |
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 |
9 |
['bryangingechen', 'euprunin', 'github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'leanprover-community-mathlib4-bot'] |
nobody |
3-11765 3 days ago |
25-34050 25 days ago |
29-50893 29 days |
26640 |
euprunin author:euprunin |
chore: golf Data/ using `grind` |
|
t-data |
13/96 |
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 |
20 |
['euprunin', 'github-actions', 'grunweg', 'leanprover-bot', 'leanprover-community-mathlib4-bot'] |
nobody |
3-11687 3 days ago |
7-42870 7 days ago |
30-45028 30 days |
26840 |
oliver-butterley author:oliver-butterley |
feat(Mathlib/Dynamics/BirkhoffSum/Average): add 3 BirkhoffAverage lemmas |
- `birkhoffAverage_add`
- `birkhoffAverage_neg`
- `birkhoffAverage_sub`
- `birkhoffSum_add'`
- `birkhoffSum_neg`
- `birkhoffSum_sub`
Co-authored-by: Lua Viana Reis
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-dynamics
|
34/1 |
Mathlib/Dynamics/BirkhoffSum/Average.lean,Mathlib/Dynamics/BirkhoffSum/Basic.lean |
2 |
5 |
['ADedecker', 'estradilua', 'github-actions', 'oliver-butterley'] |
nobody |
3-5639 3 days ago |
3-70638 3 days ago |
26-3535 26 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 |
9 |
['github-actions', 'joelriou', 'robin-carlier'] |
nobody |
2-85680 2 days ago |
2-85680 2 days ago |
20-29373 20 days |
27641 |
FormulaRabbit81 author:FormulaRabbit81 |
feat: Proof of relative compactness implies tightness of a set of measures (Easy direction of Prokhorov's theorem). |
PR proving the easy direction of Prokhorov's theorem. I am not sure about the naming conventions and any comments are appreciated.
---
[](https://gitpod.io/from-referrer/)
|
large-import
new-contributor
t-measure-probability
|
260/1 |
Mathlib/Analysis/SpecificLimits/Basic.lean,Mathlib/Data/ENNReal/Operations.lean,Mathlib/MeasureTheory/Measure/ProbabilityMeasure.lean,Mathlib/MeasureTheory/Measure/Tight.lean |
4 |
3 |
['FormulaRabbit81', 'github-actions', 'themathqueen'] |
nobody |
2-77699 2 days ago |
3-11297 3 days ago |
3-62538 3 days |
27681 |
sgouezel author:sgouezel |
feat: one implication of portmanteau theorem for countably generated filters |
Also weaken a few assumptions in this file from metric spaces to metrizable spaces.
---
[](https://gitpod.io/from-referrer/)
|
t-measure-probability |
48/8 |
Mathlib/MeasureTheory/Measure/Portmanteau.lean |
1 |
1 |
['github-actions'] |
nobody |
2-71305 2 days ago |
2-71313 2 days ago |
2-71363 2 days |
27682 |
FernandoChu author:FernandoChu |
Chore: Added `vecAppend_empty` lemma |
Added the `vecAppend_empty`.
|
t-data
new-contributor
|
5/0 |
Mathlib/Data/Fin/VecNotation.lean |
1 |
1 |
['github-actions'] |
nobody |
2-67738 2 days ago |
2-67738 2 days ago |
2-67949 2 days |
27549 |
Ruben-VandeVelde author:Ruben-VandeVelde |
feat: Submodule.smul_one_eq_span |
Co-authored-by: Aaron Hill
Co-authored-by: Austin Letson
Co-authored-by: Matej Penciak
---
From FLT
[](https://gitpod.io/from-referrer/)
|
FLT
t-algebra
easy
label:t-algebra$ |
3/0 |
Mathlib/Algebra/Algebra/Operations.lean |
1 |
3 |
['github-actions', 'ocfnash'] |
nobody |
2-63882 2 days ago |
5-62986 5 days ago |
5-63034 5 days |
27556 |
kebekus author:kebekus |
feat: analyticity of harmonic functions, Part I |
If `f : ℂ → ℝ` is harmonic at `x`, show that `∂f/∂1 - I • ∂f/∂I` is complex-analytic at `x`.
As soon as PR #9598 (feat(Analysis/Complex): HasPrimitives on disc) is merged, I will extend this result to show that `f` itself is locally the real part of a holomorphic function, and hence real-analytic.
---
[](https://gitpod.io/from-referrer/)
|
t-analysis |
66/0 |
Mathlib.lean,Mathlib/Analysis/InnerProductSpace/Harmonic/Analytic.lean |
2 |
3 |
['github-actions', 'kebekus', 'sgouezel'] |
nobody |
2-51674 2 days ago |
5-54194 5 days ago |
5-54239 5 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'] |
eric-wieser assignee:eric-wieser |
2-47165 2 days ago |
83-38711 2 months ago |
83-40264 83 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'] |
dagurtomas assignee:dagurtomas |
2-47163 2 days ago |
71-27326 2 months ago |
71-27377 71 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'] |
alexjbest assignee:alexjbest |
2-47162 2 days ago |
58-51718 1 month ago |
59-62065 59 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'] |
ericrbg assignee:ericrbg |
2-47159 2 days ago |
13-37835 13 days ago |
33-84393 33 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'] |
joelriou assignee:joelriou |
2-47158 2 days ago |
27-66858 27 days ago |
40-31341 40 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'] |
dagurtomas assignee:dagurtomas |
2-47157 2 days ago |
44-74340 1 month ago |
44-74384 44 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'] |
ericrbg assignee:ericrbg |
2-47155 2 days ago |
36-40836 1 month ago |
36-85595 36 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'] |
ericrbg assignee:ericrbg |
2-47154 2 days ago |
31-17478 1 month ago |
31-17741 31 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'] |
eric-wieser assignee:eric-wieser |
2-47151 2 days ago |
23-51552 23 days ago |
23-51598 23 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'] |
b-mehta assignee:b-mehta |
2-47150 2 days ago |
21-84353 21 days ago |
21-84397 21 days |
27664 |
pechersky author:pechersky |
feat(Topology,Analysis): discrete topology metric space and normed groups |
Explicit construction of the discrete topology metric space and normed groups where `dist x y = 1` for all `x != y`
Provide PseudoMetricSpace, MetricSpace, Seminormed(Add)Group, and Normed(Add)Group constructions
---
[](https://gitpod.io/from-referrer/)
|
t-topology |
137/0 |
Mathlib/Analysis/Normed/Group/Basic.lean,Mathlib/Topology/MetricSpace/Basic.lean,Mathlib/Topology/MetricSpace/Pseudo/Constructions.lean |
3 |
1 |
['github-actions'] |
nobody |
2-47101 2 days ago |
3-18002 3 days ago |
3-17996 3 days |
27697 |
BoltonBailey author:BoltonBailey |
chore(Data/Fintype): use `univ` instead of `Fintype.elems` |
A short PR to keep the API consistent with its surroundings.
---
[](https://gitpod.io/from-referrer/)
|
t-data |
2/2 |
Mathlib/Data/Fintype/Defs.lean |
1 |
1 |
['github-actions', 'vihdzp'] |
nobody |
2-43331 2 days ago |
2-47210 2 days ago |
2-47256 2 days |
27238 |
alreadydone author:alreadydone |
feat(Algebra): IsDomain R[X] ↔ IsDomain R ∧ IsCancelAdd R |
---
- [x] depends on: #27241
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebra
label:t-algebra$ |
138/4 |
Counterexamples.lean,Counterexamples/PolynomialIsDomain.lean,Mathlib/Algebra/Group/Defs.lean,Mathlib/Algebra/Group/Opposite.lean,Mathlib/Algebra/GroupWithZero/Defs.lean,Mathlib/Algebra/GroupWithZero/TransferInstance.lean,Mathlib/Algebra/Opposites.lean,Mathlib/Algebra/Polynomial/Basic.lean,Mathlib/RingTheory/Polynomial/Opposites.lean |
9 |
6 |
['alreadydone', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
2-41863 2 days ago |
2-42231 2 days ago |
3-12845 3 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 |
146 |
['YaelDillies', 'copilot-pull-request-reviewer', 'eric-wieser', 'github-actions', 'plp127', 'quangvdao', 'tannerduve'] |
nobody |
2-38998 2 days ago |
45-63784 1 month ago |
55-82866 55 days |
27015 |
vihdzp author:vihdzp |
feat: `aleph` and `beth` are normal functions |
By using `Order.IsNormal`, we can state (and use!) these results directly, instead of having to go through `ord`.
---
- [x] depends on: #26900
[](https://gitpod.io/from-referrer/)
|
|
58/40 |
Mathlib/Order/ConditionallyCompleteLattice/Indexed.lean,Mathlib/Order/IsNormal.lean,Mathlib/SetTheory/Cardinal/Aleph.lean |
3 |
4 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
2-38616 2 days ago |
2-38640 2 days ago |
2-41411 2 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
|
174/0 |
Mathlib.lean,Mathlib/Computability/PrimrecFilter.lean |
2 |
65 |
['DavidJWebb', 'github-actions', 'grunweg'] |
nobody |
2-37742 2 days ago |
2-37938 2 days ago |
30-51854 30 days |
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 |
7 |
['JovanGerb', 'eric-wieser', 'github-actions'] |
kim-em assignee:kim-em |
2-30502 2 days ago |
30-25994 30 days ago |
30-26046 30 days |
27703 |
vihdzp author:vihdzp |
feat: `le_of_forall_ne` |
This form of `le_of_forall_lt` is a bit nicer when working with nimbers; they're minimum excludents, so to prove `a ≤ b` you have to prove `b` can't be equal to any smaller `a`!
---
[](https://gitpod.io/from-referrer/)
|
t-order
easy
|
7/0 |
Mathlib/Order/Basic.lean |
1 |
1 |
['github-actions'] |
nobody |
2-30122 2 days ago |
2-39356 2 days ago |
2-39358 2 days |
27705 |
yonggyuchoimath author:yonggyuchoimath |
feat(RingTheory.Ideal.Height): add trivial cases |
feat: add trivial cases of Ideal.Height
---
This PR updates `RingTheory.Ideal.Height`, which adds two lemmas `Ideal.height_of_subsingleton` and `Ideal.height_bot_eq_zero`. These compute the height of (any) ideal in a zero commutative ring, and the height of the zero ideal in a nonzero commutative ring. |
new-contributor
t-algebra
label:t-algebra$ |
9/0 |
Mathlib/RingTheory/Ideal/Height.lean |
1 |
5 |
['erdOne', 'github-actions', 'yonggyuchoimath'] |
nobody |
2-25312 2 days ago |
2-36766 2 days ago |
2-36811 2 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 |
419/84 |
Mathlib/Tactic/Widget/Conv.lean,MathlibTest/conv?.lean |
2 |
4 |
['bryangingechen', 'github-actions', 'plp127'] |
bryangingechen assignee:bryangingechen |
2-20848 2 days ago |
48-21614 1 month ago |
48-21659 48 days |
27712 |
kim-em author:kim-em |
chore: remove old irrelevant attributes in Logic/Basic |
This PR removes some attributes from Logic/Basic that appear to have no effect on Mathlib. |
t-logic |
0/2 |
Mathlib/Logic/Basic.lean |
1 |
4 |
['github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot'] |
nobody |
2-19257 2 days ago |
2-19257 2 days ago |
2-24156 2 days |
27162 |
themathqueen author:themathqueen |
feat(Analysis/InnerProductSpace/Positive): `U.starProjection ≤ V.starProjection` iff `U ≤ V` |
For star projections `p` and `q`, `p ≤ q` iff `p ∘ q = p`, so then a corollary is: `U.starProjection ≤ V.starProjection` iff `U ≤ V`.
---
- [x] depends on: #25910
- [x] depends on: #27619
[](https://gitpod.io/from-referrer/)
|
|
37/0 |
Mathlib/Analysis/InnerProductSpace/Positive.lean |
1 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
2-8001 2 days ago |
2-10419 2 days ago |
2-11211 2 days |
27534 |
PierreQuinton author:PierreQuinton |
Add `LawfulPreorder` |
Adds lawful infima and suprema type classes.
A preorder with lawful suprema: whenever a set has a least upper bound, `sSup` returns a least upper bound for that set.
A preorder with lawful infima: whenever a set has a greatest lower bound, `sInf` returns a greastest lower bound for that set.
---
[](https://gitpod.io/from-referrer/)
|
t-order |
121/8 |
Mathlib.lean,Mathlib/Order/CompleteLattice/Defs.lean,Mathlib/Order/LawfulSupInf.lean |
3 |
11 |
['PierreQuinton', 'github-actions', 'vihdzp'] |
nobody |
2-4697 2 days ago |
5-61453 5 days ago |
5-61488 5 days |
27720 |
peabrainiac author:peabrainiac |
feat(CategoryTheory/Adjunction): lemmas on adjoint quadruples |
Lemmas about adjoint quadruples `L ⊣ F ⊣ G ⊣ R` where some of the functors are fully faithful:
* If `F` and `R` are fully faithful, the components of the induced natural transformation `G ⟶ L`
are epic iff the components of the natural transformation `F ⟶ R` are monic.
* If `L` and `G` are fully faithful, the components of the induced natural transformation `L ⟶ G`
are epic iff the components of the natural transformation `R ⟶ F` are monic.
A variant of the first case appears as proposition 2.7 on the nlab [here](https://ncatlab.org/nlab/show/cohesive+topos); the second case is dual.
From [lean-orbifolds](https://github.com/peabrainiac/lean-orbifolds/blob/d599ff5f39aa831e8fa79b2f2fa7178b36bcbafd/Orbifolds/ForMathlib/Quadruple.lean).
---
Continued / revived from #24667. |
t-category-theory |
178/0 |
Mathlib.lean,Mathlib/CategoryTheory/Adjunction/Quadruple.lean,Mathlib/CategoryTheory/Adjunction/Triple.lean,Mathlib/CategoryTheory/Category/Basic.lean,Mathlib/CategoryTheory/EpiMono.lean |
5 |
2 |
['github-actions', 'peabrainiac'] |
nobody |
2-4451 2 days ago |
2-5868 2 days ago |
2-6575 2 days |
27383 |
euprunin author:euprunin |
chore: replace `omega` with `grind` in `Algebra/` theorems/lemmas where applicable |
Motivation: `grind` subsumes `omega`, which is expected to be deprecated. |
t-algebra label:t-algebra$ |
225/225 |
Mathlib/Algebra/AddConstMap/Basic.lean,Mathlib/Algebra/BigOperators/Fin.lean,Mathlib/Algebra/CharP/Defs.lean,Mathlib/Algebra/ContinuedFractions/Computation/Approximations.lean,Mathlib/Algebra/ContinuedFractions/Computation/TerminatesIffRat.lean,Mathlib/Algebra/CubicDiscriminant.lean,Mathlib/Algebra/GCDMonoid/Nat.lean,Mathlib/Algebra/GeomSum.lean,Mathlib/Algebra/Group/Defs.lean,Mathlib/Algebra/Group/Int/Even.lean,Mathlib/Algebra/Group/Nat/Range.lean,Mathlib/Algebra/GroupWithZero/Basic.lean,Mathlib/Algebra/GroupWithZero/Units/Basic.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/Basic.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/EnoughInjectives.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/EnoughProjectives.lean,Mathlib/Algebra/Homology/DerivedCategory/Fractions.lean,Mathlib/Algebra/Homology/Embedding/Basic.lean,Mathlib/Algebra/Homology/Embedding/Boundary.lean,Mathlib/Algebra/Homology/Embedding/CochainComplex.lean,Mathlib/Algebra/Homology/Embedding/Connect.lean,Mathlib/Algebra/Homology/ExactSequence.lean,Mathlib/Algebra/Homology/HomotopyCategory/HomComplex.lean,Mathlib/Algebra/Homology/HomotopyCategory/HomComplexShift.lean,Mathlib/Algebra/Homology/HomotopyCategory/Pretriangulated.lean,Mathlib/Algebra/Homology/HomotopyCategory/ShiftSequence.lean,Mathlib/Algebra/Homology/HomotopyCategory/ShortExact.lean,Mathlib/Algebra/Homology/TotalComplexShift.lean,Mathlib/Algebra/Lie/LieTheorem.lean,Mathlib/Algebra/Lie/Nilpotent.lean,Mathlib/Algebra/Lie/Sl2.lean,Mathlib/Algebra/Lie/Weights/Chain.lean,Mathlib/Algebra/Lie/Weights/Killing.lean,Mathlib/Algebra/Lie/Weights/RootSystem.lean,Mathlib/Algebra/Module/LinearMap/End.lean,Mathlib/Algebra/MvPolynomial/Degrees.lean,Mathlib/Algebra/Order/Antidiag/Nat.lean,Mathlib/Algebra/Order/Floor/Ring.lean,Mathlib/Algebra/Order/Group/Basic.lean,Mathlib/Algebra/Order/Group/Int/Sum.lean,Mathlib/Algebra/Order/Group/Unbundled/Int.lean,Mathlib/Algebra/Order/GroupWithZero/Unbundled/Basic.lean,Mathlib/Algebra/Order/Monoid/Unbundled/Pow.lean,Mathlib/Algebra/Order/Ring/Int.lean,Mathlib/Algebra/Order/Ring/Unbundled/Rat.lean,Mathlib/Algebra/Polynomial/AlgebraMap.lean,Mathlib/Algebra/Polynomial/Degree/IsMonicOfDegree.lean,Mathlib/Algebra/Polynomial/Derivative.lean,Mathlib/Algebra/Polynomial/FieldDivision.lean,Mathlib/Algebra/Polynomial/Laurent.lean,Mathlib/Algebra/Polynomial/Module/Basic.lean,Mathlib/Algebra/Polynomial/OfFn.lean,Mathlib/Algebra/Polynomial/Sequence.lean,Mathlib/Algebra/Polynomial/UnitTrinomial.lean,Mathlib/Algebra/Ring/Divisibility/Lemmas.lean,Mathlib/Algebra/Squarefree/Basic.lean,Mathlib/Algebra/Vertex/VertexOperator.lean |
57 |
18 |
['euprunin', 'github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'leanprover-community-mathlib4-bot'] |
nobody |
2-822 2 days ago |
2-840 2 days ago |
9-34614 9 days |
27339 |
pechersky author:pechersky |
chore(RingTheory/Laurent): use WithZero.exp to golf statements and proofs about valuation on K((X)) |
Done as part of refactor of Valued in #27314. This PR does not change any definitions. Instead, uses `WithZero.exp` instead of coercion + Multiplicative.ofAdd. And some helper simp lemmas about valuations of RatFunc vis a vis LaurentSeries.
---
[](https://gitpod.io/from-referrer/)
|
tech debt
t-algebra
t-number-theory
label:t-algebra$ |
78/77 |
Mathlib/FieldTheory/RatFunc/AsPolynomial.lean,Mathlib/RingTheory/LaurentSeries.lean,Mathlib/Topology/Algebra/Valued/WithVal.lean |
3 |
1 |
['github-actions'] |
Vierkantor assignee:Vierkantor |
1-85478 1 day ago |
10-64257 10 days ago |
11-21853 11 days |
27738 |
ChrisHughes24 author:ChrisHughes24 |
feat(Rat): Decidable instance for IsSquare |
---
[](https://gitpod.io/from-referrer/)
|
t-data |
3/0 |
Mathlib/Data/Rat/Lemmas.lean |
1 |
1 |
['github-actions'] |
nobody |
1-83946 1 day ago |
1-83950 1 day ago |
1-83998 1 day |
27735 |
kebekus author:kebekus |
feat: mean value property of complex differentiable functions on the complex plane |
As an immediate application of the Cauchy integral formula, establish the mean value property of complex-differentiable functions on the complex plane. Fix a typo in the docstrings of `Mathlib/Analysis/Complex/CauchyIntegral.lean` and remove one unnecessary type cast.
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.
TODO: As soon as PR https://github.com/leanprover-community/mathlib4/pull/9598 (feat(Analysis/Complex): HasPrimitives on disc) is merged, extend this to harmonic functions.
---
[](https://gitpod.io/from-referrer/)
|
t-analysis |
99/5 |
Mathlib.lean,Mathlib/Analysis/Complex/CauchyIntegral.lean,Mathlib/Analysis/Complex/MeanValue.lean,Mathlib/MeasureTheory/Integral/CircleAverage.lean |
4 |
1 |
['github-actions'] |
nobody |
1-83863 1 day ago |
1-83863 1 day ago |
2-312 2 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'] |
Vierkantor assignee:Vierkantor |
1-79122 1 day ago |
54-1447 1 month ago |
54-2385 54 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'] |
dwrensha assignee:dwrensha |
1-79121 1 day ago |
69-1141 2 months ago |
69-1192 69 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'] |
chrisflav assignee:chrisflav |
1-79120 1 day ago |
28-8084 28 days ago |
65-47657 65 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'] |
Vierkantor assignee:Vierkantor |
1-79118 1 day ago |
35-71750 1 month ago |
40-68758 40 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'] |
jcommelin assignee:jcommelin |
1-79117 1 day ago |
41-50472 1 month ago |
41-50514 41 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'] |
ericrbg assignee:ericrbg |
1-79116 1 day ago |
36-50937 1 month ago |
36-50982 36 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'] |
kbuzzard assignee:kbuzzard |
1-79115 1 day ago |
30-31662 30 days ago |
30-31708 30 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'] |
awainverse assignee:awainverse |
1-79114 1 day ago |
27-59793 27 days ago |
27-59839 27 days |
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'] |
mariainesdff assignee:mariainesdff |
1-79113 1 day ago |
15-19303 15 days ago |
27-58190 27 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 |
935/0 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/DepRewrite.lean,MathlibTest/depRewrite.lean |
4 |
6 |
['Vtec234', 'github-actions', 'kmill', 'plp127'] |
eric-wieser assignee:eric-wieser |
1-79112 1 day ago |
26-11831 26 days ago |
26-11882 26 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'] |
riccardobrasca assignee:riccardobrasca |
1-79111 1 day ago |
19-16612 19 days ago |
19-16693 19 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'] |
dagurtomas assignee:dagurtomas |
1-79109 1 day ago |
19-7086 19 days ago |
19-7156 19 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'] |
Vierkantor assignee:Vierkantor |
1-79108 1 day ago |
18-62384 18 days ago |
18-62379 18 days |
27305 |
eric-wieser author:eric-wieser |
feat: instances for `ZeroHom` and `OneHom` |
This is motivated by wanting to write some lemmas about how the def in #27272 behaves on addition and scalar multiplcation, which requires these operations to first be defined.
This shows that `ZeroHom` forms an `AddCommGroup` and `Module`, as well as analogous intermediate statements and `OneHom` results.
---
- [x] depends on: #27318
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
188/8 |
Mathlib/Algebra/Group/Hom/Basic.lean,Mathlib/Algebra/Group/Hom/Instances.lean,Mathlib/Algebra/GroupWithZero/Action/Defs.lean,Mathlib/Algebra/GroupWithZero/Action/Hom.lean,Mathlib/Algebra/Module/Hom.lean,Mathlib/GroupTheory/GroupAction/DomAct/Basic.lean |
6 |
3 |
['eric-wieser', 'github-actions', 'mathlib4-dependent-issues-bot'] |
ericrbg assignee:ericrbg |
1-79107 1 day ago |
9-43695 9 days ago |
9-43679 9 days |
27741 |
ShreckYe author:ShreckYe |
feat(Algebra/ModEq): add the `IsTrans` instance for `AddCommGroup.ModEq` |
The `trans` theorem is present for `AddCommGroup.ModEq` but there is no type class instance, while a similar instance is present for `Int.ModEq`, so I guess it should be missing. |
new-contributor
t-algebra
easy
label:t-algebra$ |
3/0 |
Mathlib/Algebra/ModEq.lean |
1 |
2 |
['ShreckYe', 'github-actions'] |
nobody |
1-78947 1 day ago |
1-78948 1 day ago |
1-79322 1 day |
27742 |
ChrisHughes24 author:ChrisHughes24 |
feat(Nat/nth): inequalities about Nat.nth |
---
[](https://gitpod.io/from-referrer/)
|
t-data |
58/0 |
Mathlib/Data/Nat/Nth.lean |
1 |
1 |
['github-actions'] |
nobody |
1-78394 1 day ago |
1-78402 1 day ago |
1-78448 1 day |
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 |
787/600 |
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 |
29 |
['ADedecker', 'PatrickMassot', 'YaelDillies', 'b-mehta', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
1-76711 1 day ago |
1-76735 1 day ago |
64-83876 64 days |
27716 |
kim-em author:kim-em |
chore: factor out lemmas from `LinearOrder ℚ` |
|
maintainer-merge
t-algebra
label:t-algebra$ |
26/16 |
Mathlib/Algebra/Order/Ring/Unbundled/Rat.lean |
1 |
3 |
['github-actions', 'grunweg'] |
nobody |
1-75433 1 day ago |
1-75433 1 day ago |
2-19891 2 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* |
t-algebraic-topology
large-import
|
253/7 |
Mathlib/AlgebraicTopology/SimplexCategory/GeneratorsRelations/NormalForms.lean |
1 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
1-75178 1 day ago |
1-75178 1 day ago |
51-4942 51 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-algebraic-topology |
118/5 |
Mathlib/AlgebraicTopology/SimplexCategory/Basic.lean,Mathlib/AlgebraicTopology/SimplicialSet/Degenerate.lean |
2 |
2 |
['github-actions', 'joelriou'] |
nobody |
1-75163 1 day ago |
1-75163 1 day ago |
44-84640 44 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 (at least after forgetting the topology), 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-algebraic-topology |
258/0 |
Mathlib.lean,Mathlib/AlgebraicTopology/SimplicialObject/II.lean |
2 |
3 |
['github-actions', 'joelriou', 'mathlib4-dependent-issues-bot'] |
nobody |
1-74965 1 day ago |
1-74965 1 day ago |
17-6660 17 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 |
8 |
['alreadydone', 'github-actions', 'grunweg', 'wwylele'] |
j-loreaux assignee:j-loreaux |
1-73329 1 day ago |
19-46157 19 days ago |
19-47499 19 days |
27552 |
Equilibris author:Equilibris |
chore: make typevec.arrow work over different universes |
This will be needed to allow `M.corec` to be generic across universes
---
[](https://gitpod.io/from-referrer/)
|
t-data
new-contributor
|
16/10 |
Mathlib/Data/TypeVec.lean |
1 |
3 |
['Equilibris', 'github-actions', 'plp127'] |
nobody |
1-72616 1 day ago |
5-60427 5 days ago |
5-60472 5 days |
27309 |
kckennylau author:kckennylau |
feat(CategoryTheory): a presheaf on `CostructuredArrow F d` can be extended to a presheaf on `C` |
---
Zulip: [#Is there code for X? > over category via a functor](https://leanprover.zulipchat.com/#narrow/channel/217875-Is-there-code-for-X.3F/topic/over.20category.20via.20a.20functor/with/529574191)
[](https://gitpod.io/from-referrer/)
|
t-category-theory |
218/0 |
Mathlib.lean,Mathlib/CategoryTheory/Comma/Presheaf/LeftExtension.lean |
2 |
3 |
['erdOne', 'github-actions', 'robin-carlier'] |
erdOne assignee:erdOne |
1-72366 1 day ago |
12-62327 12 days ago |
12-62378 12 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 |
6 |
['b-mehta', 'github-actions'] |
b-mehta assignee:b-mehta |
1-71164 1 day ago |
49-83970 1 month ago |
49-83954 49 days |
25952 |
101damnations author:101damnations |
feat(RepresentationTheory/Homological/GroupHomology/Functoriality): the degree 1 part of the corestriction-coinflation exact sequence when the subgroup acts trivially |
Given a normal subgroup `S` of `G` and a `G`-representation `A` on which `S` acts trivially, this PR defines the short complex
`H₁(S, A) ⟶ H₁(G, A) ⟶ H₁(G ⧸ S, A)` induced by the natural inclusion `S → G` and projection `G → G / S`. We show it is exact and that the righthand map is an epimorphism.
---
- [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 version at #22654* |
maintainer-merge
t-algebra
label:t-algebra$ |
142/2 |
Mathlib/RepresentationTheory/Homological/GroupCohomology/Functoriality.lean,Mathlib/RepresentationTheory/Homological/GroupHomology/Functoriality.lean |
2 |
n/a |
['101damnations', 'github-actions', 'kbuzzard', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
1-70898 1 day ago |
unknown |
unknown |
25966 |
b-reinke author:b-reinke |
feat(GroupTheory/FreeGroup): add predicate for reduced words |
This PR adds the predicate of reduced words `IsReduced` in the construction of free groups. It is shown that `reduce` and `toWord` produce reduced words.
This is done in preparation for the theory of cyclically reduced words.
Upstreamed from the [EquationalTheories](https://github.com/teorth/equational_theories) project.
---
This PR continues the work from #23368.
Original PR: https://github.com/leanprover-community/mathlib4/pull/23368 |
maintainer-merge
t-algebra
label:t-algebra$ |
82/0 |
Mathlib/GroupTheory/FreeGroup/Basic.lean,Mathlib/GroupTheory/FreeGroup/Reduce.lean |
2 |
35 |
['YaelDillies', 'b-reinke', 'github-actions', 'vlad902'] |
nobody |
1-67956 1 day ago |
1-78417 1 day ago |
45-69271 45 days |
27270 |
EtienneC30 author:EtienneC30 |
chore: turn WithLp into a structure |
Turn `WithLp` into a one field structure, as was suggested many times on Zulip and discussed here: https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/defeq.20abuse.20in.20.60WithLp.60/near/526234806.
Here is what this PR does:
- The instances on `WithLp p α` which were defeq to those on `α` (algebraic instances, topology, uniformity, bornology) are now pulled back from `α` along `WithLp.equiv p α`. A few declarations are added to ease the process, such as versions of `WithLp.equiv` as a homeomorphism or a uniform isomorphism.
- It introduces some definitions to equip `α × β` with the Lp distance, and similarly for `Π i, α i`. This is then used to define relevant instances on type synonyms, such as for matrix norms.
- The PR fixes all the defeq abuses (which break obviously).
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-analysis
|
756/399 |
Archive/Hairer.lean,Mathlib.lean,Mathlib/Algebra/Module/ZLattice/Covolume.lean,Mathlib/Analysis/Analytic/WithLp.lean,Mathlib/Analysis/CStarAlgebra/Matrix.lean,Mathlib/Analysis/Calculus/ContDiff/WithLp.lean,Mathlib/Analysis/Calculus/FDeriv/WithLp.lean,Mathlib/Analysis/InnerProductSpace/PiL2.lean,Mathlib/Analysis/InnerProductSpace/ProdL2.lean,Mathlib/Analysis/InnerProductSpace/Spectrum.lean,Mathlib/Analysis/Matrix.lean,Mathlib/Analysis/Normed/Algebra/TrivSqZeroExt.lean,Mathlib/Analysis/Normed/Algebra/UnitizationL1.lean,Mathlib/Analysis/Normed/Lp/LpEquiv.lean,Mathlib/Analysis/Normed/Lp/MeasurableSpace.lean,Mathlib/Analysis/Normed/Lp/PiLp.lean,Mathlib/Analysis/Normed/Lp/ProdLp.lean,Mathlib/Analysis/Normed/Lp/WithLp.lean,Mathlib/Analysis/Quaternion.lean,Mathlib/Analysis/RCLike/Inner.lean,Mathlib/Analysis/SpecialFunctions/Gaussian/FourierTransform.lean,Mathlib/Combinatorics/Additive/AP/Three/Behrend.lean,Mathlib/Geometry/Manifold/Instances/Icc.lean,Mathlib/Geometry/Manifold/Instances/Real.lean,Mathlib/LinearAlgebra/Matrix/PosDef.lean,Mathlib/LinearAlgebra/Matrix/Spectrum.lean,Mathlib/MeasureTheory/Measure/Haar/InnerProductSpace.lean,Mathlib/MeasureTheory/Measure/Haar/OfBasis.lean,Mathlib/MeasureTheory/Measure/Lebesgue/VolumeOfBalls.lean,Mathlib/NumberTheory/NumberField/CanonicalEmbedding/Basic.lean,Mathlib/NumberTheory/NumberField/Ideal/Asymptotics.lean |
31 |
5 |
['eric-wieser', 'github-actions', 'leanprover-community-bot-assistant'] |
nobody |
1-67439 1 day ago |
1-72549 1 day ago |
14-23993 14 days |
27751 |
Vierkantor author:Vierkantor |
feat: `erw?` supports all arguments that `erw` does |
This PR teaches `erw?` how to deal with multiple arguments and how to rewrite at a hypothesis, so that it can be used everywhere that `erw` can. (And ideally `erw` can then be removed from those places.)
In addition to the new tests, I picked a few places in the library to run as test cases with more complicated terms (but `extract_goals` didn't really work there...)
---
[](https://gitpod.io/from-referrer/)
|
t-meta |
146/15 |
Mathlib/Tactic/ErwQuestion.lean,MathlibTest/ErwQuestion.lean |
2 |
1 |
['github-actions'] |
nobody |
1-66511 1 day ago |
1-66590 1 day ago |
1-66574 1 day |
27419 |
grunweg author:grunweg |
chore(IntegrableOn): generalise one more section to enorms |
---
[](https://gitpod.io/from-referrer/)
|
carleson
maintainer-merge
t-measure-probability
|
139/96 |
Mathlib/Analysis/MellinTransform.lean,Mathlib/Analysis/SpecialFunctions/ImproperIntegrals.lean,Mathlib/Analysis/SpecialFunctions/Integrability/Basic.lean,Mathlib/Analysis/SpecialFunctions/Integrals/LogTrigonometric.lean,Mathlib/MeasureTheory/Integral/ExpDecay.lean,Mathlib/MeasureTheory/Integral/IntegrableOn.lean,Mathlib/MeasureTheory/Integral/IntervalIntegral/Basic.lean,Mathlib/MeasureTheory/Integral/IntervalIntegral/FundThmCalculus.lean,Mathlib/MeasureTheory/Integral/IntervalIntegral/Periodic.lean,Mathlib/MeasureTheory/Measure/Lebesgue/Integral.lean,Mathlib/NumberTheory/AbelSummation.lean,Mathlib/NumberTheory/LSeries/SumCoeff.lean |
12 |
8 |
['YaelDillies', 'github-actions', 'grunweg', 'sgouezel'] |
YaelDillies assignee:YaelDillies |
1-65194 1 day ago |
1-65194 1 day ago |
9-3030 9 days |
27754 |
Parcly-Taxel author:Parcly-Taxel |
feat: `finCycle` as iterated `finRotate` |
Originally used in #25786, but eventually discovered to be unnecessary. |
t-logic |
26/5 |
Mathlib/Logic/Equiv/Fin/Rotate.lean |
1 |
1 |
['github-actions'] |
nobody |
1-62733 1 day ago |
1-62738 1 day ago |
1-62792 1 day |
25786 |
Parcly-Taxel author:Parcly-Taxel |
feat: IMO 2001 Q4 |
|
IMO
maintainer-merge
|
106/0 |
Archive.lean,Archive/Imo/Imo2001Q4.lean |
2 |
11 |
['Parcly-Taxel', 'dwrensha', 'github-actions', 'leanprover-community-bot-assistant'] |
dwrensha assignee:dwrensha |
1-62216 1 day ago |
1-62216 1 day ago |
49-6688 49 days |
27757 |
mbkybky author:mbkybky |
feat(RingTheory): `IsTensorProduct` versions of the lemmas about tensoring with a flat module preserves injections |
Add some lemmas about `IsTensorProduct` and the `IsTensorProduct` versions of the lemmas about tensoring with a flat module preserves injections.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
220/19 |
Mathlib/RingTheory/Flat/Basic.lean,Mathlib/RingTheory/IsTensorProduct.lean |
2 |
1 |
['github-actions'] |
nobody |
1-61488 1 day ago |
1-61676 1 day ago |
1-61728 1 day |
27691 |
bryangingechen author:bryangingechen |
ci: rebuild until `lake build --no-build` succeeds |
This should hopefully help with the CI failing in the cache verification step in the Post-Build job, as recently observed on various PRs in: [#mathlib4 > Failing CI @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Failing.20CI/near/530878203).
Also adds `-v` to the `lake build --no-build` steps as well as `-wfail` to the `Archive` and `Counterexamples` build steps (cf. #19633 for the latter).
The log output will be long, so we use [GitHub's log grouping feature](https://docs.github.com/en/actions/reference/workflows-and-actions/workflow-commands#grouping-log-lines) to make the logs easier to navigate.
---
[](https://gitpod.io/from-referrer/)
|
CI |
143/36 |
.github/build.in.yml,.github/workflows/bors.yml,.github/workflows/build.yml,.github/workflows/build_fork.yml,scripts/README.md,scripts/lake-build-with-retry.sh |
6 |
10 |
['bryangingechen', 'github-actions', 'grunweg', 'kim-em', 'tydeu'] |
nobody |
1-58405 1 day ago |
1-63037 1 day ago |
2-11674 2 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 |
13 |
['eric-wieser', 'github-actions', 'joelriou', 'leanprover-community-bot-assistant'] |
nobody |
1-57866 1 day ago |
1-66304 1 day ago |
32-5427 32 days |
27762 |
plp127 author:plp127 |
chore(AbstractCompletion): universe polymorphism |
---
[](https://gitpod.io/from-referrer/)
|
t-topology |
17/16 |
Mathlib/Topology/UniformSpace/AbstractCompletion.lean |
1 |
1 |
['github-actions'] |
nobody |
1-56542 1 day ago |
1-56612 1 day ago |
1-56661 1 day |
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 ∈ 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
|
327/30 |
Mathlib.lean,Mathlib/Order/Hom/Lattice.lean,Mathlib/Order/Nucleus.lean,Mathlib/Order/Sublocale.lean,Mathlib/Order/Synonym.lean,docs/references.bib |
6 |
91 |
['Bergschaf', 'YaelDillies', 'b-mehta', 'bryangingechen', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'xhalo32'] |
bryangingechen assignee:bryangingechen |
1-55986 1 day ago |
55-46602 1 month ago |
69-26023 69 days |
27763 |
j-loreaux author:j-loreaux |
feat: define morphism type `StarMonoidHom` |
This defines star-preserving monoid homomorphisms between star monoids.
The primary motivation for these morphisms is to provide a target type for morphisms which induce a corresponding morphism between the unitary groups in a star monoid.
Without this type, there is no concrete type for [unitary.map](https://leanprover-community.github.io/mathlib4_docs/Mathlib/Algebra/Star/Unitary.html#unitary.map) and we end up resorting to morphisms *classes* instead, which is suboptimal.
See [Zulip](https://leanprover.zulipchat.com/#narrow/channel/113489-new-members/topic/.E2.9C.94.20Golfing.20matrix.20group.20coercion/near/528000462) for the problem which motivated the creation of this type.
---
In a follow-up PR, I will redefine `unitary.map` so that it takes a `StarMonoidHom` as an argument and also outputs a `StarMonoidHom`. I will also add `unitary.mapEquiv` for a version which does the same for `StarMulEquiv`.
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
335/0 |
Mathlib.lean,Mathlib/Algebra/Star/MonoidHom.lean |
2 |
1 |
['github-actions'] |
nobody |
1-54723 1 day ago |
1-54760 1 day ago |
1-54774 1 day |
27696 |
pechersky author:pechersky |
feat(Padic/WithVal): WithVal v is isomorphic to Q_p as fields and uniform spaces |
On the way to a topological ring equiv
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-number-theory
label:t-algebra$ |
187/0 |
Mathlib.lean,Mathlib/NumberTheory/Padics/PadicNumbers.lean,Mathlib/NumberTheory/Padics/WithVal.lean |
3 |
1 |
['github-actions'] |
nobody |
1-52110 1 day ago |
2-48040 2 days ago |
2-48038 2 days |
27708 |
vihdzp author:vihdzp |
feat: unions and intersections of ordinals are ordinals |
As well as a bonus result `IsTransitive.empty_mem`.
---
[](https://gitpod.io/from-referrer/)
|
t-set-theory |
58/16 |
Mathlib/SetTheory/ZFC/Basic.lean,Mathlib/SetTheory/ZFC/Ordinal.lean |
2 |
3 |
['b-mehta', 'github-actions', 'vihdzp'] |
nobody |
1-48484 1 day ago |
2-30876 2 days ago |
2-30921 2 days |
27786 |
staroperator author:staroperator |
feat(GroupTheory/Finiteness): `AddMonoid.FG ℕ` and `AddGroup.FG ℤ` |
Note: [`Module.Finite.self`](https://leanprover-community.github.io/mathlib4_docs/Mathlib/RingTheory/Finiteness/Basic.html#Module.Finite.self) gives equivalent results as `Module.Finite ℕ ℕ` and `Module.Finite ℤ ℤ`. But there is no instance from `Module.Finite` to `AddMonoid.FG` (there is one converse, [AddMonoid.FG.to_moduleFinite_nat](https://leanprover-community.github.io/mathlib4_docs/Mathlib/RingTheory/Finiteness/Defs.html#AddMonoid.FG.to_moduleFinite_nat)).
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
10/0 |
Mathlib/GroupTheory/Finiteness.lean |
1 |
1 |
['github-actions'] |
nobody |
1-46324 1 day ago |
1-46331 1 day ago |
1-46378 1 day |
27787 |
staroperator author:staroperator |
feat(GroupTheory/Finiteness): instance `Monoid.fg_of_group_fg` |
This makes one direction of `Group.fg_iff_monoid_fg` an instance.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
5/0 |
Mathlib/GroupTheory/Finiteness.lean |
1 |
1 |
['github-actions'] |
nobody |
1-46222 1 day ago |
1-46228 1 day ago |
1-46275 1 day |
27449 |
kckennylau author:kckennylau |
feat(Topology): finite dimensional vector space over locally compact complete space is locally compact |
*From the 2025 Local Class Field Theory Workshop.*
---
[](https://gitpod.io/from-referrer/)
|
maintainer-merge
t-topology
|
18/0 |
Mathlib/Topology/Algebra/Module/FiniteDimension.lean |
1 |
7 |
['ADedecker', 'github-actions', 'kbuzzard', 'kckennylau', 'mariainesdff'] |
nobody |
1-45968 1 day ago |
4-62443 4 days ago |
5-10802 5 days |
27511 |
Nebula691 author:Nebula691 |
feat(Algebra/QuadraticAlgebra) : Define Quadratic Algebra |
co-authored-by : Edison Xie
co-authored-by : Kenny Lau
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-algebra
label:t-algebra$ |
418/0 |
Mathlib.lean,Mathlib/Algebra/QuadraticAlgebra.lean |
2 |
59 |
['Whysoserioushah', 'eric-wieser', 'github-actions', 'kckennylau'] |
nobody |
1-45554 1 day ago |
6-62291 6 days ago |
6-62336 6 days |
27094 |
smorel394 author:smorel394 |
feat(Algebra.Category.FGModuleCat.Colimits): the category of finitely generated modules has finite colimits |
Prove that the forgetful functor from `FGModuleCat k` to `ModuleCat k` creates finite colimits, and hence that `FGModuleCat k` has finite colimits.
- [ ] depends on: #27092
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
70/0 |
Mathlib.lean,Mathlib/Algebra/Category/FGModuleCat/Colimits.lean |
2 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
1-44824 1 day ago |
2-49867 2 days ago |
2-51045 2 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'] |
kim-em assignee:kim-em |
1-42213 1 day ago |
19-57480 19 days ago |
29-56865 29 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'] |
Vierkantor assignee:Vierkantor |
1-42212 1 day ago |
77-3570 2 months ago |
126-82521 126 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'] |
mattrobball assignee:mattrobball |
1-42211 1 day ago |
70-71259 2 months ago |
87-56280 87 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'] |
kmill assignee:kmill |
1-42210 1 day ago |
67-33761 2 months ago |
67-33815 67 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'] |
joneugster assignee:joneugster |
1-42207 1 day ago |
50-79616 1 month ago |
50-79599 50 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'] |
ericrbg assignee:ericrbg |
1-42206 1 day ago |
48-72771 1 month ago |
48-76475 48 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'] |
ericrbg assignee:ericrbg |
1-42206 1 day ago |
40-15090 1 month ago |
40-22840 40 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'] |
alreadydone assignee:alreadydone |
1-42205 1 day ago |
39-4400 1 month ago |
39-4382 39 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'] |
ericrbg assignee:ericrbg |
1-42202 1 day ago |
36-80750 1 month ago |
38-49288 38 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'] |
kim-em assignee:kim-em |
1-42201 1 day ago |
34-68751 1 month ago |
34-68798 34 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'] |
adomani assignee:adomani |
1-42201 1 day ago |
17-85161 17 days ago |
26-35054 26 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'] |
Vierkantor assignee:Vierkantor |
1-42200 1 day ago |
24-45592 24 days ago |
24-45640 24 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'] |
bryangingechen assignee:bryangingechen |
1-42198 1 day ago |
17-35234 17 days ago |
17-35278 17 days |
27355 |
alreadydone author:alreadydone |
feat(Algebra): annihilator of fg module over PID is ann of some element |
Live coding at *Formalizing Class Field Theory* for the finite case of the normal basis theorem
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
50/0 |
Mathlib/Algebra/Module/PID.lean,Mathlib/RingTheory/Ideal/Maps.lean |
2 |
6 |
['alreadydone', 'github-actions', 'kckennylau'] |
jcommelin assignee:jcommelin |
1-42195 1 day ago |
10-53221 10 days ago |
10-53205 10 days |
27715 |
dupuisf author:dupuisf |
feat(CStarAlgebra): `a => a ^ p` is operator monotone for `p ∈ Icc 0 1` |
This PR shows that `a => a ^ p` is operator monotone for `p ∈ Icc 0 1`, i.e. that `CFC.nnrpow`, `CFC.rpow` and `CFC.sqrt` are monotone, using the integral representation for the power function.
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-analysis
|
307/12 |
Mathlib/Algebra/Algebra/Spectrum/Quasispectrum.lean,Mathlib/Analysis/Normed/Algebra/Spectrum.lean,Mathlib/Analysis/SpecialFunctions/ContinuousFunctionalCalculus/Rpow/IntegralRepresentation.lean,Mathlib/Topology/ContinuousOn.lean |
4 |
1 |
['github-actions'] |
nobody |
1-40681 1 day ago |
1-40686 1 day ago |
1-40670 1 day |
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'] |
chrisflav assignee:chrisflav |
1-37643 1 day ago |
58-46020 1 month ago |
58-46071 58 days |
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'] |
alexjbest assignee:alexjbest |
1-37642 1 day ago |
57-42551 1 month ago |
57-42609 57 days |
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 |
357/2 |
Mathlib/Algebra/Order/Archimedean/Class.lean,Mathlib/RingTheory/HahnSeries/Lex.lean |
2 |
14 |
['ScottCarnahan', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'wwylele'] |
alreadydone assignee:alreadydone |
1-37641 1 day ago |
21-28255 21 days ago |
39-60848 39 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'] |
joneugster assignee:joneugster |
1-37640 1 day ago |
39-62440 1 month ago |
43-33690 43 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'] |
mattrobball assignee:mattrobball |
1-37639 1 day ago |
43-31671 1 month ago |
43-31715 43 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'] |
ADedecker assignee:ADedecker |
1-37638 1 day ago |
21-72288 21 days ago |
41-11228 41 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'] |
Vierkantor assignee:Vierkantor |
1-37634 1 day ago |
26-2918 26 days ago |
26-2965 26 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 |
91/37 |
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'] |
alexjbest assignee:alexjbest |
1-37630 1 day ago |
19-83957 19 days ago |
19-83985 19 days |
27304 |
jano-wol author:jano-wol |
feat: invariant dual submodules define Lie ideals |
Invariant dual submodules define Lie ideals
---
PR shows that Invariant dual submodules define Lie ideals.
This work is part of the framework: https://github.com/orgs/leanprover-community/projects/17
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
358/0 |
Mathlib.lean,Mathlib/Algebra/Lie/Weights/InvariantSubmoduleLieIdeal.lean,Mathlib/Algebra/Lie/Weights/Killing.lean,Mathlib/Algebra/Lie/Weights/RootSystem.lean |
4 |
1 |
['github-actions'] |
jcommelin assignee:jcommelin |
1-37628 1 day ago |
12-75567 12 days ago |
12-75614 12 days |
27380 |
chrisflav author:chrisflav |
feat(Category/Ring): `Algebra.IsPushout` iff `CategoryTheory.IsPushout` |
In particular, `RingHom.IsStableUnderBaseChange P` iff `(RingHom.toMorphismProperty P).IsStableUnderCobaseChange`.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
49/0 |
Mathlib/Algebra/Category/Ring/Constructions.lean,Mathlib/RingTheory/IsTensorProduct.lean,Mathlib/RingTheory/RingHomProperties.lean |
3 |
1 |
['github-actions'] |
joelriou assignee:joelriou |
1-37627 1 day ago |
10-8003 10 days ago |
10-7986 10 days |
26693 |
euprunin author:euprunin |
chore: golf Computability/ using `grind` |
|
maintainer-merge
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 |
8 |
['euprunin', 'github-actions', 'grunweg', 'leanprover-bot', 'leanprover-community-mathlib4-bot'] |
YaelDillies assignee:YaelDillies |
1-36049 1 day ago |
1-36049 1 day ago |
29-52686 29 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 |
279/11 |
Mathlib.lean,Mathlib/Analysis/InnerProductSpace/GramSchmidtOrtho.lean,Mathlib/Topology/VectorBundle/GramSchmidtOrtho.lean,scripts/noshake.json |
4 |
67 |
['faenuccio', 'github-actions', 'grunweg', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'sgouezel'] |
sgouezel assignee:sgouezel |
1-36039 1 day ago |
16-35118 16 days ago |
16-42668 16 days |
27711 |
wwylele author:wwylele |
feat(Algebra/Order): Add Add/Mul/Linear equiv versions of toLex/ofLex |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
84/30 |
Mathlib.lean,Mathlib/Algebra/Order/Group/Equiv.lean,Mathlib/Algebra/Order/GroupWithZero/Lex.lean,Mathlib/Algebra/Order/Module/Equiv.lean |
4 |
7 |
['github-actions', 'pechersky', 'wwylele'] |
nobody |
1-32181 1 day ago |
2-20986 2 days ago |
2-25567 2 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.
Note: the import increase happens in a leaf file `Mathlib.RingTheory.FractionalIdeal.Extended`
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebra
label:t-algebra$ |
190/5 |
Mathlib/RingTheory/DedekindDomain/Ideal/Lemmas.lean,Mathlib/RingTheory/FractionalIdeal/Extended.lean,Mathlib/RingTheory/Localization/Basic.lean |
3 |
2 |
['github-actions', 'leanprover-community-bot-assistant'] |
nobody |
1-30858 1 day ago |
1-31067 1 day ago |
14-80362 14 days |
27792 |
kim-em author:kim-em |
feat: plumbing version of ClearExcept tactic |
|
t-meta |
17/8 |
Mathlib/Tactic/ClearExcept.lean |
1 |
1 |
['github-actions'] |
nobody |
1-30671 1 day ago |
1-30685 1 day ago |
1-30732 1 day |
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
t-number-theory
label:t-algebra$ |
89/3 |
Mathlib/RingTheory/DedekindDomain/Factorization.lean,Mathlib/RingTheory/DedekindDomain/Ideal/Basic.lean,Mathlib/RingTheory/DedekindDomain/Ideal/Lemmas.lean,Mathlib/RingTheory/Ideal/Operations.lean,Mathlib/RingTheory/Ideal/Over.lean |
5 |
2 |
['github-actions', 'leanprover-community-bot-assistant'] |
nobody |
1-29390 1 day ago |
1-29413 1 day ago |
19-362 19 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 |
173/2 |
Mathlib/NumberTheory/NumberField/Ideal/KummerDedekind.lean,Mathlib/NumberTheory/RamificationInertia/Basic.lean,Mathlib/RingTheory/AdjoinRoot.lean,Mathlib/RingTheory/DedekindDomain/Ideal/Lemmas.lean,Mathlib/RingTheory/Ideal/Over.lean |
5 |
5 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'xroblot'] |
nobody |
1-27385 1 day ago |
1-29058 1 day ago |
0-50 50 seconds |
27055 |
wwylele author:wwylele |
feat(RingTheory): add HahnSeries.trunc |
---
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/)
|
maintainer-merge
t-algebra
label:t-algebra$ |
53/0 |
Mathlib/RingTheory/HahnSeries/Addition.lean,Mathlib/RingTheory/HahnSeries/Basic.lean |
2 |
6 |
['Ruben-VandeVelde', 'ScottCarnahan', 'github-actions', 'kbuzzard', 'wwylele'] |
nobody |
1-25158 1 day ago |
7-7089 7 days ago |
20-21582 20 days |
27794 |
xroblot author:xroblot |
feat(RingTheory): add `symm_apply_eq` and `eq_symm_apply` for `RingEquiv` |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
easy
label:t-algebra$ |
6/0 |
Mathlib/Algebra/Ring/Equiv.lean |
1 |
1 |
['github-actions'] |
nobody |
1-23637 1 day ago |
1-23650 1 day ago |
1-23695 1 day |
27442 |
artie2000 author:artie2000 |
feat(RingTheory/NonUnitalSubsemiring): add Aesop rules for `-(x * y)` subsemiring membership |
The Aesop rule `mul_mem` doesn't decompose goals of the form `-x * y ∈ s` or `x * -y ∈ s` in the absence of `neg_mem` because these expressions simplify to `-(x * y) ∈ s`.
---
[](https://gitpod.io/from-referrer/)
|
maintainer-merge
t-algebra
label:t-algebra$ |
22/1 |
Mathlib/RingTheory/NonUnitalSubsemiring/Defs.lean |
1 |
20 |
['Vierkantor', 'YaelDillies', 'artie2000', 'eric-wieser', 'github-actions'] |
YaelDillies assignee:YaelDillies |
0-60400 16 hours ago |
3-53776 3 days ago |
7-15345 7 days |
27622 |
ShreckYe author:ShreckYe |
feat(Analysis/SpecialFunctions/Trigonometric): add the missing `tan_sub` and `tan_sub'` functions for both real and complex numbers |
While working on some proofs, I found that the `tan_sub` theorems are missing, while there are the corresponding`sin_sub` and `cos_sub` theorems. So I'd like to propose adding these for `tan`. |
new-contributor
t-analysis
|
38/0 |
Mathlib/Analysis/SpecialFunctions/Trigonometric/Arctan.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Complex.lean |
2 |
4 |
['Ruben-VandeVelde', 'ShreckYe', 'github-actions', 'leanprover-community-bot-assistant'] |
nobody |
1-19567 1 day ago |
1-19584 1 day ago |
3-55774 3 days |
27790 |
pechersky author:pechersky |
feat(Topology): `IsDenseInducing.isUniformInducing_extend` |
extending along a uniform inducing function with another uniform inducing function with dense ranges of both
creates a uniform inducing extension
golfs a proof in #27696
and discussed in https://leanprover.zulipchat.com/#narrow/channel/217875-Is-there-code-for-X.3F/topic/isUniformInducing_extension
---
[](https://gitpod.io/from-referrer/)
|
t-topology |
62/0 |
Mathlib/Topology/DenseEmbedding.lean,Mathlib/Topology/UniformSpace/AbstractCompletion.lean,Mathlib/Topology/UniformSpace/Completion.lean,Mathlib/Topology/UniformSpace/UniformEmbedding.lean |
4 |
2 |
['github-actions', 'plp127'] |
nobody |
1-17106 1 day ago |
1-38188 1 day ago |
1-38220 1 day |
27163 |
pechersky author:pechersky |
feat(Topology/ValuativeRel): of and to basis of compatible valuations |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-topology
t-number-theory
label:t-algebra$ |
106/20 |
Mathlib/RingTheory/Valuation/ValuativeRel.lean,Mathlib/Topology/Algebra/Valued/ValuativeRel.lean |
2 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
1-13997 1 day ago |
1-16421 1 day ago |
17-54476 17 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$ |
74/1 |
Mathlib/RingTheory/Valuation/ValuativeRel.lean,Mathlib/Topology/Algebra/Valued/ValuativeRel.lean |
2 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
alreadydone assignee:alreadydone |
1-13140 1 day ago |
1-16547 1 day ago |
24-59282 24 days |
27492 |
euprunin author:euprunin |
chore: further golf some previously `grind` golfed proofs |
Replaces #27431, #27426, #27408 and #27404.
It is probably safer to go with local `grind [t1, t2, …]` for now and leave global `@[grind =, etc.] theorem t1 …` annotations for later. I guess the local `grind [t1, t2, …]` uses can help guide which `t1`, `t2`, etc are worth to annotate "globally". |
|
8/30 |
Mathlib/Algebra/BigOperators/Group/Finset/Basic.lean,Mathlib/LinearAlgebra/LinearPMap.lean,Mathlib/RingTheory/DividedPowers/Basic.lean,Mathlib/Topology/EMetricSpace/BoundedVariation.lean |
4 |
6 |
['github-actions', 'kim-em', 'leanprover-bot', 'mathlib-bors'] |
nobody |
1-10072 1 day ago |
1-10093 1 day ago |
7-30886 7 days |
27577 |
bjornsolheim author:bjornsolheim |
feat(Data/Fin/Tuple): lemmas on appending finite sequences |
Prove simple results regarding appending and de-appending of finite sequences.
Used to define conical combinations and the conical hull (subsequent PR).
---
[](https://gitpod.io/from-referrer/)
|
t-data
new-contributor
|
42/0 |
Mathlib/Data/Fin/Tuple/Basic.lean |
1 |
19 |
['YaelDillies', 'bjornsolheim', 'eric-wieser', 'github-actions'] |
nobody |
1-9613 1 day ago |
1-9613 1 day ago |
2-54998 2 days |
27802 |
euprunin author:euprunin |
chore(Algebra): golf using the `have […] := by grind` pattern |
|
t-algebra label:t-algebra$ |
4/9 |
Mathlib/Algebra/CharP/Defs.lean,Mathlib/Algebra/Lie/Engel.lean,Mathlib/Algebra/Order/BigOperators/Ring/Finset.lean |
3 |
1 |
['github-actions'] |
nobody |
1-8925 1 day ago |
1-8934 1 day ago |
1-8983 1 day |
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 |
1-8518 1 day ago |
19-65607 19 days ago |
19-65589 19 days |
27777 |
grunweg author:grunweg |
chore(Algebra/Group/Support): rename primed lemmas to match naming convention |
`mulSupport_inv` should be called `mulSupport_fun_inv`, according to the [naming convention](https://leanprover-community.github.io/contribute/naming.html#unexpanded-and-expanded-forms-of-functions),
similarly for the other lemmas.
Unfortunately, there is no good tooling yet for renames `A -> B` and `B -> C`.
---
[](https://gitpod.io/from-referrer/)
|
maintainer-merge
t-algebra
label:t-algebra$ |
42/28 |
Mathlib/Algebra/BigOperators/Finprod.lean,Mathlib/Algebra/Group/Indicator.lean,Mathlib/Algebra/Group/Support.lean,Mathlib/Algebra/GroupWithZero/Indicator.lean,Mathlib/LinearAlgebra/RootSystem/Base.lean,Mathlib/MeasureTheory/Function/SimpleFunc.lean,Mathlib/MeasureTheory/Function/StronglyMeasurable/Basic.lean,Mathlib/RingTheory/HahnSeries/Addition.lean,Mathlib/RingTheory/HahnSeries/Basic.lean,Mathlib/Topology/Algebra/Support.lean,Mathlib/Topology/LocallyFinsupp.lean |
11 |
4 |
['YaelDillies', 'github-actions', 'grunweg'] |
nobody |
1-8322 1 day ago |
1-8322 1 day ago |
1-41865 1 day |
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 |
5 |
['github-actions', 'grunweg', 'loefflerd', 'riccardobrasca', 'xroblot'] |
nobody |
1-6767 1 day ago |
37-66676 1 month ago |
37-66709 37 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$ |
705/634 |
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 |
3 |
['github-actions', 'leanprover-community-bot-assistant'] |
joelriou assignee:joelriou |
1-6510 1 day ago |
2-7672 2 days ago |
43-40992 43 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
maintainer-merge
t-category-theory
|
178/64 |
Mathlib.lean,Mathlib/CategoryTheory/Noetherian.lean,Mathlib/CategoryTheory/Subobject/ArtinianObject.lean,Mathlib/CategoryTheory/Subobject/NoetherianObject.lean |
4 |
13 |
['github-actions', 'javra', 'joelriou', 'robin-carlier'] |
robin-carlier assignee:robin-carlier |
1-4022 1 day ago |
1-12719 1 day ago |
21-46498 21 days |
25002 |
YaelDillies author:YaelDillies |
chore(Finsupp): move order properties under `Order` |
---
[](https://gitpod.io/from-referrer/)
|
large-import |
360/326 |
Mathlib.lean,Mathlib/Algebra/Group/Finsupp.lean,Mathlib/Algebra/MvPolynomial/Basic.lean,Mathlib/Algebra/Order/Floor/Div.lean,Mathlib/Data/Finsupp/Ext.lean,Mathlib/Data/Finsupp/Multiset.lean,Mathlib/Data/Finsupp/Order.lean,Mathlib/Data/Finsupp/PWO.lean,Mathlib/Data/Finsupp/Pointwise.lean,Mathlib/Data/Finsupp/SMulWithZero.lean,Mathlib/Data/Finsupp/Single.lean,Mathlib/Data/Finsupp/Weight.lean,Mathlib/Data/List/ToFinsupp.lean,Mathlib/Data/Nat/Choose/Multinomial.lean,Mathlib/Data/Nat/Factorization/Defs.lean,Mathlib/Order/Preorder/Finsupp.lean |
16 |
7 |
['bryangingechen', 'github-actions', 'leanprover-community-bot-assistant'] |
bryangingechen assignee:bryangingechen |
1-3022 1 day ago |
6-84500 6 days ago |
43-65777 43 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/73 |
Mathlib/Data/List/ProdSigma.lean,Mathlib/Tactic/Simproc/ExistsAndEq.lean,MathlibTest/Simproc/ExistsAndEq.lean |
3 |
10 |
['JovanGerb', 'github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'leanprover-community-mathlib4-bot', 'mathlib4-merge-conflict-bot', 'vasnesterov'] |
kmill assignee:kmill |
1-2507 1 day ago |
1-2530 1 day ago |
25-74670 25 days |
27805 |
euprunin author:euprunin |
chore(Algebra/Order): golf `mem_piAntidiag` and `trichotomy_of_mul_eq_mul` using `grind` |
|
maintainer-merge
t-algebra
label:t-algebra$ |
3/3 |
Mathlib/Algebra/Order/Antidiag/Pi.lean,Mathlib/Algebra/Order/Monoid/Unbundled/Basic.lean |
2 |
2 |
['github-actions', 'grunweg'] |
nobody |
0-86179 23 hours ago |
0-86179 23 hours ago |
1-1883 1 day |
27803 |
euprunin author:euprunin |
chore(Algebra/ContinuedFractions): golf `fib_le_of_contsAux_b`, `sub_convs_eq` and `abs_sub_convs_le` using `grind` |
|
maintainer-merge
t-algebra
label:t-algebra$ |
3/20 |
Mathlib/Algebra/ContinuedFractions/Computation/Approximations.lean |
1 |
2 |
['github-actions', 'grunweg'] |
nobody |
0-86157 23 hours ago |
0-86157 23 hours ago |
1-2211 1 day |
27801 |
euprunin author:euprunin |
chore(Algebra/Order+Polynomial): golf entire `sub_self_div_two`, `div_two_sub_self`, `add_two_le_iff_lt_of_even_sub` and `natDegree_pos_of_nextCoeff_ne_zero` using `grind` |
|
maintainer-merge
t-algebra
label:t-algebra$ |
4/9 |
Mathlib/Algebra/Order/Field/Basic.lean,Mathlib/Algebra/Order/Ring/Int.lean,Mathlib/Algebra/Polynomial/Degree/Lemmas.lean |
3 |
2 |
['github-actions', 'grunweg'] |
nobody |
0-86134 23 hours ago |
0-86134 23 hours ago |
1-9420 1 day |
27640 |
Louddy author:Louddy |
feat(RatFunc): liftAlgebra and rank |
Add analogous results from `FractionRing` in the special case of `RatFunc`. This is needed as `RatFunc` is a one-field-struct. The first three are scoped instances lifting structure from `K[X]` to `RatFunc K`. Our application is two results stating that with appropriate context, the rank of `RatFunc K` over `RatFunc k` is the rank of `K` over `k`.
- `RatFunc.liftAlgebra` ([`FractionRing`version](https://leanprover-community.github.io/mathlib4_docs/Mathlib/RingTheory/Localization/FractionRing.html#FractionRing.liftAlgebra))
- `RatFunc.isScalarTower_liftAlgebra` ([`FractionRing` version](https://leanprover-community.github.io/mathlib4_docs/Mathlib/RingTheory/Localization/FractionRing.html#FractionRing.isScalarTower_liftAlgebra))
- `RatFunc.faithfulSMul'` ([`FractionRing` version](https://leanprover-community.github.io/mathlib4_docs/Mathlib/RingTheory/Localization/FractionRing.html#FractionRing.instFaithfulSMul))
- `RatFunc.rank_ratFunc_ratFunc` (mathlib has a version for [`FractionRing`](https://leanprover-community.github.io/mathlib4_docs/Mathlib/RingTheory/Algebraic/Integral.html#Algebra.IsAlgebraic.rank_fractionRing_polynomial) but we use the version for [`IsFractionRing`](https://leanprover-community.github.io/mathlib4_docs/Mathlib/RingTheory/Algebraic/Integral.html#Algebra.IsAlgebraic.rank_of_isFractionRing) combined with `rank_polynomial_polynomial`.)
- `RatFunc.finrank_ratFunc_ratFunc`
The first three are declared as scoped instances of `RatFunc`. This creates a conflict with the current `LaurentSeries` file. To fix this, I have refactored to use the algebra instance coming from `RatFunc.liftAlgebra` instead of the `coeAlgHom` map defined in `LaurentSeries`.
This has two main effects:
- It simplifies the file.
- The instance `RatFunc.instCoePolynomial` does not need to be hidden anymore.
Looking forward to feedback!
Xavier
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$ |
76/106 |
Mathlib/FieldTheory/RatFunc/Basic.lean,Mathlib/RingTheory/LaurentSeries.lean |
2 |
1 |
['github-actions'] |
nobody |
0-84476 23 hours ago |
0-84476 23 hours ago |
1-1662 1 day |
27807 |
grunweg author:grunweg |
chore: mark Polynomial.differential fun_prop |
And remove a superfluous `local fun_prop` tag: Complex.continuous_abs is already marked fun_prop.
---
[](https://gitpod.io/from-referrer/)
|
easy |
1/3 |
Mathlib/Analysis/Calculus/Deriv/Polynomial.lean,Mathlib/NumberTheory/Transcendental/Lindemann/AnalyticalPart.lean |
2 |
1 |
['github-actions'] |
nobody |
0-83033 23 hours ago |
0-83100 23 hours ago |
0-83085 23 hours |
27809 |
euprunin author:euprunin |
chore(Algebra/Module): golf `eq_zero_of_ofSpanSingleton_apply_self` using `grind […]` |
|
t-algebra label:t-algebra$ |
4/12 |
Mathlib/Algebra/Module/CharacterModule.lean |
1 |
1 |
['github-actions'] |
nobody |
0-81939 22 hours ago |
0-82394 22 hours ago |
0-82440 22 hours |
27804 |
euprunin author:euprunin |
chore(Algebra/Polynomial): golf `coeff_mul_natTrailingDegree_add_natTrailingDegree` and `div_eq_quo_add_sum_rem_div` using `grind [Finset.*]` |
|
maintainer-merge
t-algebra
label:t-algebra$ |
3/13 |
Mathlib/Algebra/Polynomial/Degree/TrailingDegree.lean,Mathlib/Algebra/Polynomial/PartialFractions.lean |
2 |
2 |
['github-actions', 'grunweg'] |
nobody |
0-81899 22 hours ago |
0-86167 23 hours ago |
1-2044 1 day |
27781 |
euprunin author:euprunin |
chore(Topology/Algebra): golf `prod_subset` using `grind [Set.*]` |
|
t-topology |
2/4 |
Mathlib/Topology/Algebra/Nonarchimedean/Basic.lean |
1 |
1 |
['github-actions'] |
nobody |
0-81797 22 hours ago |
1-47190 1 day ago |
1-47242 1 day |
27628 |
EtienneC30 author:EtienneC30 |
feat(ProbabilityTheory): a new predicate HasLaw |
Introduce a predicate `HasLaw X μ P` stating that the random variable `X` has law `μ` under the measure `P`. This is expressed as `P.map X = μ`. We also require `X` to be `P`-almost-everywhere measurable to avoid pathological cases.
from BrownianMotion
---
[](https://gitpod.io/from-referrer/)
|
t-measure-probability |
128/0 |
Mathlib.lean,Mathlib/Probability/HasLaw.lean |
2 |
6 |
['DavidLedvinka', 'EtienneC30', 'github-actions', 'kex-y'] |
nobody |
0-81730 22 hours ago |
3-85207 3 days ago |
3-85191 3 days |
27728 |
euprunin author:euprunin |
chore(Data/Complex): golf `norm_exp_sub_sum_le_norm_mul_exp` using `grind [Finset.*]` |
|
t-data
maintainer-merge
|
1/4 |
Mathlib/Data/Complex/Exponential.lean |
1 |
2 |
['github-actions', 'grunweg'] |
nobody |
0-81689 22 hours ago |
1-76389 1 day ago |
2-1836 2 days |
27563 |
euprunin author:euprunin |
chore(Topology/EMetricSpace/BoundedVariation): golf `add_le_union` using `grind [Finset.*]` |
|
t-topology |
2/13 |
Mathlib/Topology/EMetricSpace/BoundedVariation.lean |
1 |
1 |
['github-actions'] |
nobody |
0-81646 22 hours ago |
5-47858 5 days ago |
5-47908 5 days |
27561 |
euprunin author:euprunin |
chore(Topology/EMetricSpace/BoundedVariation): golf `add_point` using `grind [Finset.*]` |
|
t-topology |
5/26 |
Mathlib/Topology/EMetricSpace/BoundedVariation.lean |
1 |
1 |
['github-actions'] |
nobody |
0-81624 22 hours ago |
5-49224 5 days ago |
5-49274 5 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'] |
MichaelStollBayreuth assignee:MichaelStollBayreuth |
0-80765 22 hours ago |
79-84759 2 months ago |
79-84740 79 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'] |
kim-em assignee:kim-em |
0-80760 22 hours ago |
73-23034 2 months ago |
73-23089 73 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'] |
joelriou assignee:joelriou |
0-80756 22 hours ago |
27-67024 27 days ago |
27-71301 27 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'] |
kim-em assignee:kim-em |
0-80753 22 hours ago |
47-73441 1 month ago |
47-73490 47 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'] |
riccardobrasca assignee:riccardobrasca |
0-80750 22 hours ago |
28-67941 28 days ago |
42-74121 42 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'] |
kim-em assignee:kim-em |
0-80745 22 hours ago |
45-52049 1 month ago |
45-52032 45 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'] |
j-loreaux assignee:j-loreaux |
0-80740 22 hours ago |
38-83273 1 month ago |
38-83319 38 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$ |
120/37 |
Mathlib/LinearAlgebra/BilinearForm/Properties.lean,Mathlib/RingTheory/DedekindDomain/Different.lean,Mathlib/RingTheory/Trace/Basic.lean |
3 |
1 |
['github-actions'] |
adomani assignee:adomani |
0-80738 22 hours ago |
38-2345 1 month ago |
38-2395 38 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'] |
awainverse assignee:awainverse |
0-80737 22 hours ago |
30-2911 30 days ago |
30-2962 30 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'] |
kbuzzard assignee:kbuzzard |
0-80733 22 hours ago |
25-50114 25 days ago |
25-50378 25 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 |
8 |
['github-actions', 'grunweg', 'mathlib4-dependent-issues-bot', 'michaellee94'] |
ocfnash assignee:ocfnash |
0-80731 22 hours ago |
22-55530 22 days ago |
22-70201 22 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'] |
adomani assignee:adomani |
0-80728 22 hours ago |
20-8208 20 days ago |
20-40065 20 days |
27308 |
xyzw12345 author:xyzw12345 |
feat(LinearAlgebra/SymmetricAlgebra): IsSymmetricAlgebra |
This PR continues the work from #24602.
Original PR: https://github.com/leanprover-community/mathlib4/pull/24602 |
t-algebra label:t-algebra$ |
78/0 |
Mathlib/LinearAlgebra/SymmetricAlgebra/Basic.lean,Mathlib/LinearAlgebra/SymmetricAlgebra/Basis.lean |
2 |
1 |
['github-actions'] |
mattrobball assignee:mattrobball |
0-80726 22 hours ago |
12-65324 12 days ago |
12-65377 12 days |
27439 |
Vierkantor author:Vierkantor |
chore(*): review 2024-04-01 adaptation notes |
There are three kinds of adaptation notes from the changes on 2024-04-01.
One about `erw` "blowing up"; this referred to a backwards compatibility flag that was already removed long ago (#14064). So this can just be deleted.
A few about needing to use `symm` before `ext` fires: this is because `apply` failing to unify when mixing very general limit definitions and very specific operations for equalizers/pullbacks. I propose we fix this by unfolding the terms manually in an `intro` type ascription. In the longer term we should consider instead specializing the limit lemmas to these specific shapes.
A few about `aesop` not working. This has the same underlying cause, due to `ext` not applying, so it now looks like `intro s (m : _ --> _) x; aesop`. Same specializing of the limit lemmas may be useful here.
---
[](https://gitpod.io/from-referrer/)
|
tech debt |
8/25 |
Mathlib/AlgebraicGeometry/Spec.lean,Mathlib/CategoryTheory/Limits/Shapes/KernelPair.lean,Mathlib/CategoryTheory/Limits/Shapes/Kernels.lean,Mathlib/CategoryTheory/Limits/Shapes/Products.lean |
4 |
2 |
['github-actions', 'grunweg'] |
jcommelin assignee:jcommelin |
0-80521 22 hours ago |
8-53153 8 days ago |
8-53137 8 days |
26210 |
Thmoas-Guan author:Thmoas-Guan |
feat(RingTheory): associated primes of localized module |
We prove that `Ass(S^{-1}M)` is equal to the preimage of `Ass(M)` under `Ideal.comap` if the base ring is Noetherian.
From this we conclude that every minimal prime 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$ |
79/17 |
Mathlib/RingTheory/Ideal/AssociatedPrime/Localization.lean |
1 |
17 |
['Thmoas-Guan', 'chrisflav', 'github-actions', 'mbkybky'] |
nobody |
0-78345 21 hours ago |
0-78596 21 hours ago |
28-24218 28 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
|
13/0 |
Mathlib/MeasureTheory/PiSystem.lean |
1 |
13 |
['EtienneC30', 'KiringYJ', 'github-actions', 'ocfnash'] |
nobody |
0-78181 21 hours ago |
1-64028 1 day ago |
28-51872 28 days |
27814 |
xroblot author:xroblot |
feat(FieldTheory/Galois): add `IsGalois.of_equiv_equiv` |
Assume that `E/F` is Galois and that `F ≃+* M` and `E ≃+* N` with some compatibility hypothesis, then `N/M` is Galois
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
32/0 |
Mathlib/Algebra/Polynomial/Eval/Degree.lean,Mathlib/FieldTheory/Galois/Basic.lean,Mathlib/FieldTheory/Minpoly/Field.lean,Mathlib/FieldTheory/Normal/Defs.lean |
4 |
1 |
['github-actions'] |
nobody |
0-75852 21 hours ago |
0-75858 21 hours ago |
0-75905 21 hours |
27816 |
BGuillemet author:BGuillemet |
feat(CategoryTheory/Sites/SheafOfTypes): composition of a sheaf with uliftFunctor is still a sheaf |
Prove that if a presheaf of types is a sheaf, then its composition with `uliftFunctor` is still a sheaf.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-category-theory
|
4/0 |
Mathlib/CategoryTheory/Sites/SheafOfTypes.lean |
1 |
1 |
['github-actions'] |
nobody |
0-73524 20 hours ago |
0-73560 20 hours ago |
0-73583 20 hours |
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 |
12 |
['alexkeizer', 'eric-wieser', 'github-actions', 'quangvdao'] |
nobody |
0-73311 20 hours ago |
24-29058 24 days ago |
24-29103 24 days |
27819 |
BGuillemet author:BGuillemet |
feat(CategoryTheory/Yoneda): add curried version of Yoneda lemma for heterogeneous universes, and other version of homNatIso |
Prove a curried version of `yonedaCompUliftFunctorEquiv`, ie a completely functorial version of the Yoneda lemma with heterogeneous universes. Dually, prove a curried version of `coyonedaCompUliftFunctorEquiv`, ie a completely functorial version of the coYoneda lemma with heterogeneous universes.
In addition, prove a functorial version of `FullyFaithful.natEquiv` using `coyoneda` instead of `yoneda` (previously, the only functorial version of `FullyFaithful.natEquiv` were `homNatIso`, which is written using `yoneda`).
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-category-theory
|
162/36 |
Mathlib/CategoryTheory/Yoneda.lean |
1 |
1 |
['github-actions'] |
nobody |
0-72394 20 hours ago |
0-72472 20 hours ago |
0-72473 20 hours |
27815 |
BGuillemet author:BGuillemet |
feat(CategoryTheory/Limits/Shapes/Products): add limMapPi and sigmaMapColim |
Add the canonical morphism from a limit to the product over its objects. Prove that it is a monomorphism.
Dually, add the canonical morphism to a colimit from the coproduc of its objects and prove that it is an epimorphism.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-category-theory
|
44/0 |
Mathlib/CategoryTheory/Limits/Shapes/Products.lean |
1 |
1 |
['github-actions'] |
nobody |
0-72160 20 hours ago |
0-74088 20 hours ago |
0-74114 20 hours |
27820 |
FLDutchmann author:FLDutchmann |
chore(NumberTheory/SelbergSieve): turn `BoundingSieve` into a struct |
Based on a discussion [on zulip](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/BoundingSieve.20is.20a.20class.3F.3F).
I wound up removing the custom notation as well, since not everybody was fond of it and I had some trouble getting it to work properly with structure inheritance and the corresponding coersions.
---
[](https://gitpod.io/from-referrer/)
|
t-analysis
t-number-theory
|
51/84 |
Mathlib/NumberTheory/SelbergSieve.lean |
1 |
1 |
['github-actions'] |
nobody |
0-71207 19 hours ago |
0-71230 19 hours ago |
0-71266 19 hours |
27823 |
Louddy author:Louddy |
feat(RatFunc): transcendental_X |
The variable `RatFunc.X` is transcendental of `K` in `RatFunc K`.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
10/0 |
Mathlib/FieldTheory/RatFunc/AsPolynomial.lean |
1 |
1 |
['github-actions'] |
nobody |
0-70375 19 hours ago |
0-70385 19 hours ago |
0-70431 19 hours |
27822 |
Louddy author:Louddy |
feat(RatFunc): theorems algebraMap polynomial |
Two simple lemmas about the `algebraMap` from `F[X]` to `RatFunc F`:
- A `monomial n a` is `C a * X ^ n` (here we are using `RatFunc.X` and `RatFunc.C`.)
- The algebraMap from `F[X]` to `RatFunc F` is the same as the evaluation of a polynomial `p` at `RatFunc.X`.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
easy
label:t-algebra$ |
9/0 |
Mathlib/FieldTheory/RatFunc/AsPolynomial.lean |
1 |
1 |
['github-actions'] |
nobody |
0-70363 19 hours ago |
0-70363 19 hours ago |
0-70514 19 hours |
27824 |
ChrisHughes24 author:ChrisHughes24 |
feat(Calculus): exists_gt_of_deriv_pos and variants |
---
I created a new file for this as I anticipate there will be many lemmas relating derivatives and monotonicity in future. Some lemmas relating deriviatives to monotonicity are already in mathlib and should maybe moved to the file (e.g. docs#HasDerivWithinAt.nonneg_of_monotoneOn).
I stated them in as much generality as I could, copying the generality of `HasDerivWithinAt.nonneg_of_monotoneOn`.
[](https://gitpod.io/from-referrer/)
|
t-analysis |
94/0 |
Mathlib.lean,Mathlib/Analysis/Calculus/Deriv/Order.lean |
2 |
1 |
['github-actions'] |
nobody |
0-70265 19 hours ago |
0-70276 19 hours ago |
0-70323 19 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
|
468/312 |
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 |
29 |
['FernandoChu', 'github-actions', 'joelriou', 'robin-carlier'] |
TwoFX assignee:TwoFX |
0-68372 18 hours ago |
0-68462 19 hours ago |
13-71694 13 days |
27825 |
yonggyuchoimath author:yonggyuchoimath |
feat(RingTheory/Ideal/Height): sup of ideal heights equals Krull dimension |
feat: sup of ideal heights equals Krull dimension
---
This PR adds
`Ideal.sup_height_eq_ringKrullDim`
`Ideal.sup_primeHeight_eq_ringKrullDim`
They show the suprema of heights of ideals / prime ideals are equal to the Krull dimension, when the ring is nonzero. |
new-contributor
t-algebra
label:t-algebra$ |
53/0 |
Mathlib/RingTheory/Ideal/Height.lean |
1 |
2 |
['github-actions', 'yonggyuchoimath'] |
nobody |
0-67991 18 hours ago |
0-69590 19 hours ago |
0-69639 19 hours |
27785 |
staroperator author:staroperator |
chore(Algebra/Group/Submonoid): golf `Nat.addSubmonoid_closure_one` using `simp` |
This should improve the proof readability.
---
[](https://gitpod.io/from-referrer/)
|
bench-after-CI
large-import
t-algebra
label:t-algebra$ |
5/13 |
Mathlib/Algebra/Group/Submonoid/Membership.lean,Mathlib/Algebra/Group/Submonoid/Operations.lean,Mathlib/Algebra/Order/Star/Basic.lean |
3 |
2 |
['github-actions', 'staroperator'] |
nobody |
0-67782 18 hours ago |
1-46837 1 day ago |
1-46943 1 day |
27755 |
bwangpj author:bwangpj |
feat(RepresentationTheory/Basic): direct sum of representations |
Define the `DirectSum` of a family of `Representation`s.
[Zulip thread](https://leanprover.zulipchat.com/#narrow/channel/116395-maths/topic/Representation.20Theory)
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-algebra
label:t-algebra$ |
39/0 |
Mathlib/RepresentationTheory/Basic.lean |
1 |
3 |
['bwangpj', 'github-actions', 'kbuzzard'] |
nobody |
0-67460 18 hours ago |
1-62303 1 day ago |
1-62350 1 day |
27828 |
Louddy author:Louddy |
feat(Algebra/Adjoin): singleton as aeval |
For `x : A`, elements of `Algebra.adjoin R {x}` can be represented as a polynomial of `R` evaluated at the point `x`.
This PR introduces three (3) theorems related to this:
- `adjoin_mem_exists_aeval` rewrite an element of `A` in `adjoin R {x}` as the `aeval` of some polynomial.
- `adjoin_eq_exists_aeval` rewrite an element `adjoin R {x}` as the `aeval` of some polynomial.
- `adjoin_singleton_induction`: an induction principle reducing problems over `adjoin R {x}` to problems of the form `M (⟨aeval x p, aeval_mem_adjoin_singleton R x⟩ : adjoin R {x})`.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
29/8 |
Mathlib/RingTheory/Adjoin/Polynomial.lean |
1 |
1 |
['github-actions'] |
nobody |
0-67220 18 hours ago |
0-67222 18 hours ago |
0-67275 18 hours |
27749 |
EtienneC30 author:EtienneC30 |
feat: the covariance of independent random variables is 0 and consequences |
Simplify the proofs in `Probability/Integration` and move the file in the `Independence` folder (which is the main reason for the huge diff). Use this to prove that the covariance of independent random variables is 0. Use this to golf the proof that the variance of a sum of independent random variables is the sum of their variances. Also prove that random variables on a product space are independent.
---
- [x] depends on: #27721
- [x] depends on: #27736
[](https://gitpod.io/from-referrer/)
|
large-import
t-measure-probability
|
481/402 |
Mathlib.lean,Mathlib/MeasureTheory/Function/LpSeminorm/Basic.lean,Mathlib/MeasureTheory/Measure/Prod.lean,Mathlib/Probability/Independence/Basic.lean,Mathlib/Probability/Independence/Integration.lean,Mathlib/Probability/Integration.lean,Mathlib/Probability/Moments/Basic.lean,Mathlib/Probability/Moments/Covariance.lean,Mathlib/Probability/Moments/Variance.lean |
9 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
0-65326 18 hours ago |
0-65328 18 hours ago |
0-66223 18 hours |
27674 |
EtienneC30 author:EtienneC30 |
feat: integrability in a product space |
Prove that `f : (i : ι) → X → E i` is in `Lᵖ` if and only if for all `i`, `f i` is in `Lᵖ`. Do the same for `f : X → (E × F)`. Also provide `WithLp` versions.
from BrownianMotion
---
- [x] depends on: #27721
[](https://gitpod.io/from-referrer/)
|
t-measure-probability |
276/1 |
Mathlib.lean,Mathlib/Analysis/NormedSpace/OperatorNorm/NormedSpace.lean,Mathlib/MeasureTheory/Integral/Eval/Basic.lean,Mathlib/MeasureTheory/Integral/Eval/WithLp.lean,Mathlib/Topology/MetricSpace/Injection.lean |
5 |
3 |
['RemyDegenne', 'github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
0-64656 17 hours ago |
0-64656 17 hours ago |
2-43908 2 days |
26967 |
joelriou author:joelriou |
feat(AlgebraicTopology/ModelCategory): left homotopies |
This PR studies the notion of "left homotopy" given by cylinder objects in model categories.
---
- [x] depends on: #26171
[](https://gitpod.io/from-referrer/)
|
t-algebraic-topology
t-category-theory
|
303/0 |
Mathlib.lean,Mathlib/AlgebraicTopology/ModelCategory/LeftHomotopy.lean |
2 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
robin-carlier assignee:robin-carlier |
0-63852 17 hours ago |
1-75072 1 day ago |
10-57944 10 days |
26958 |
joelriou author:joelriou |
feat(AlgebraicTopology): path objects in model categories |
This PR dualizes #26171 which was about cylinder objects.
---
- [x] depends on: #26171
[](https://gitpod.io/from-referrer/)
|
t-algebraic-topology
t-category-theory
|
335/0 |
Mathlib.lean,Mathlib/AlgebraicTopology/ModelCategory/IsCofibrant.lean,Mathlib/AlgebraicTopology/ModelCategory/PathObject.lean,Mathlib/CategoryTheory/Limits/Shapes/Pullback/CommSq.lean |
4 |
4 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
robin-carlier assignee:robin-carlier |
0-63817 17 hours ago |
1-75077 1 day ago |
11-5628 11 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 |
18 |
['RemyDegenne', 'github-actions', 'kbuzzard'] |
nobody |
0-63472 17 hours ago |
0-63544 17 hours ago |
46-7083 46 days |
26738 |
javra author:javra |
feat(AlgebraicToplogy/SimplexCategory): add notation for faces and degeneracies general truncated simplex categories |
---
[](https://gitpod.io/from-referrer/)
|
t-algebraic-topology
infinity-cosmos
|
43/32 |
Mathlib/AlgebraicTopology/SimplexCategory/Truncated.lean,Mathlib/AlgebraicTopology/SimplicialSet/HomotopyCat.lean |
2 |
4 |
['emilyriehl', 'github-actions', 'leanprover-community-bot-assistant'] |
nobody |
0-63218 17 hours ago |
0-74303 20 hours ago |
14-65306 14 days |
27707 |
FLDutchmann author:FLDutchmann |
feat(NumberTheory/SelbergSieve): define Selberg's weights and prove basic results. |
This PR continues the work from #23635.
Original PR: https://github.com/leanprover-community/mathlib4/pull/23635 |
t-analysis
t-number-theory
|
407/83 |
Mathlib/NumberTheory/Divisors.lean,Mathlib/NumberTheory/SelbergSieve.lean |
2 |
1 |
['github-actions'] |
nobody |
0-59215 16 hours ago |
0-60239 16 hours ago |
2-30746 2 days |
27637 |
Louddy author:Louddy |
feat(Subalgebra): simp lemma for algebraMap mk |
Add three lemma (two simp) for the interaction of `Subalgebra.mk` and `algebraMap`.
Let me know if you think these lemmas should be placed elsewhere.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
20/8 |
Mathlib/Algebra/Algebra/Subalgebra/Basic.lean,Mathlib/LinearAlgebra/CliffordAlgebra/Even.lean |
2 |
14 |
['Louddy', 'eric-wieser', 'github-actions'] |
nobody |
0-59081 16 hours ago |
3-61758 3 days ago |
3-61751 3 days |
27837 |
CBirkbeck author:CBirkbeck |
feat(NumberTheory/Divisors): add divisorAntidiagonal equivalence. |
---
[](https://gitpod.io/from-referrer/)
|
t-number-theory |
33/0 |
Mathlib/NumberTheory/Divisors.lean |
1 |
1 |
['github-actions'] |
nobody |
0-58834 16 hours ago |
0-58839 16 hours ago |
0-58886 16 hours |
27004 |
kbuzzard author:kbuzzard |
chore: rename doset to doubleCoset |
---
[](https://gitpod.io/from-referrer/)
I was working with these in FLT and something snapped. It's *not a word*.
|
t-algebra label:t-algebra$ |
105/41 |
Mathlib/GroupTheory/DoubleCoset.lean |
1 |
9 |
['eric-wieser', 'github-actions', 'grunweg', 'j-loreaux', 'kbuzzard'] |
nobody |
0-58756 16 hours ago |
0-58756 16 hours ago |
0-83929 23 hours |
27316 |
mans0954 author:mans0954 |
feature(Analysis/LocallyConvex/WeakDual): functional_mem_span_iff |
Sufficient and necessary conditions for a linear functional to be in the span of a finite set of linear functionals.
This result is Rudin, Functional Analysis, Second edition, Lemma 3.9 (see also Bourbaki TVS, II.6 Proposition 5).
A key application of this result is the proof that `WeakBilin.eval B` is surjective i.e. the dual of `E` with the weak topology is identified with `F`.
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-analysis
|
106/0 |
Mathlib/Analysis/LocallyConvex/WeakDual.lean,docs/references.bib |
2 |
9 |
['ADedecker', 'github-actions', 'mans0954'] |
nobody |
0-58451 16 hours ago |
4-48196 4 days ago |
9-6025 9 days |
27791 |
alreadydone author:alreadydone |
chore(Algebra/Regular): split Defs out of Basic and redefine IsCancelMul |
Redefine Is(Left/Right)CancelMul(Zero) in terms of Is(Left/Right)Regular. Defeq to the original defs except for argument explicitness/order. Part of #22997
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebra
label:t-algebra$ |
198/165 |
Archive/Imo/Imo2015Q6.lean,Mathlib.lean,Mathlib/Algebra/Group/Defs.lean,Mathlib/Algebra/Group/Prod.lean,Mathlib/Algebra/Group/TypeTags/Basic.lean,Mathlib/Algebra/Group/UniqueProds/Basic.lean,Mathlib/Algebra/GroupWithZero/Associated.lean,Mathlib/Algebra/GroupWithZero/Basic.lean,Mathlib/Algebra/GroupWithZero/Defs.lean,Mathlib/Algebra/GroupWithZero/InjSurj.lean,Mathlib/Algebra/GroupWithZero/Nat.lean,Mathlib/Algebra/GroupWithZero/Opposite.lean,Mathlib/Algebra/GroupWithZero/Regular.lean,Mathlib/Algebra/MonoidAlgebra/NoZeroDivisors.lean,Mathlib/Algebra/Order/Group/Basic.lean,Mathlib/Algebra/Order/Group/Bounds.lean,Mathlib/Algebra/Order/Group/Int/Sum.lean,Mathlib/Algebra/Order/Interval/Set/Instances.lean,Mathlib/Algebra/Order/Monoid/Unbundled/Basic.lean,Mathlib/Algebra/Order/Ring/Defs.lean,Mathlib/Algebra/Polynomial/Coeff.lean,Mathlib/Algebra/Regular/Basic.lean,Mathlib/Algebra/Regular/Defs.lean,Mathlib/Algebra/Regular/Opposite.lean,Mathlib/Algebra/Regular/Pi.lean,Mathlib/Algebra/Regular/Prod.lean,Mathlib/Algebra/Regular/SMul.lean,Mathlib/Algebra/Regular/ULift.lean,Mathlib/Algebra/Ring/Basic.lean,Mathlib/Algebra/Ring/Int/Defs.lean,Mathlib/Algebra/Ring/Regular.lean,Mathlib/Algebra/Star/Basic.lean,Mathlib/Data/Int/Interval.lean,Mathlib/Data/Int/Range.lean,Mathlib/Data/PNat/Basic.lean,Mathlib/GroupTheory/MonoidLocalization/MonoidWithZero.lean,Mathlib/Order/Interval/Finset/Box.lean,Mathlib/RingTheory/DedekindDomain/Ideal/Basic.lean,Mathlib/RingTheory/Localization/Defs.lean,Mathlib/SetTheory/Game/Impartial.lean,Mathlib/SetTheory/Nimber/Basic.lean,Mathlib/SetTheory/Nimber/Field.lean,Mathlib/Tactic/Linter/DirectoryDependency.lean,scripts/noshake.json |
44 |
2 |
['alreadydone', 'github-actions'] |
nobody |
0-58052 16 hours ago |
1-33295 1 day ago |
1-33340 1 day |
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$ |
41/9 |
Mathlib/RingTheory/Valuation/ValuativeRel.lean,Mathlib/Topology/Algebra/Valued/ValuativeRel.lean |
2 |
3 |
['Ruben-VandeVelde', 'github-actions', 'kbuzzard'] |
nobody |
0-57930 16 hours ago |
0-57940 16 hours ago |
20-11723 20 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'] |
dagurtomas assignee:dagurtomas |
0-57686 16 hours ago |
24-2116 24 days ago |
31-32813 31 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'] |
fpvandoorn assignee:fpvandoorn |
0-57686 16 hours ago |
80-8538 2 months ago |
80-8679 80 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'] |
ADedecker assignee:ADedecker |
0-57685 16 hours ago |
46-46251 1 month ago |
46-46299 46 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'] |
mariainesdff assignee:mariainesdff |
0-57684 16 hours ago |
43-67656 1 month ago |
43-67700 43 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'] |
joneugster assignee:joneugster |
0-57682 16 hours ago |
40-39609 1 month ago |
40-39657 40 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'] |
joelriou assignee:joelriou |
0-57680 16 hours ago |
23-66050 23 days ago |
23-66101 23 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'] |
mattrobball assignee:mattrobball |
0-57680 16 hours ago |
22-82851 22 days ago |
22-85193 22 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'] |
sgouezel assignee:sgouezel |
0-57679 16 hours ago |
20-58773 20 days ago |
20-61660 20 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$ |
16/6 |
Mathlib/RingTheory/DedekindDomain/AdicValuation.lean,Mathlib/Topology/Algebra/Valued/ValuedField.lean |
2 |
1 |
['github-actions'] |
mariainesdff assignee:mariainesdff |
0-57678 16 hours ago |
19-11406 19 days ago |
19-11407 19 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'] |
mariainesdff assignee:mariainesdff |
0-57677 16 hours ago |
15-61429 15 days ago |
15-61480 15 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'] |
JovanGerb assignee:JovanGerb |
0-57677 16 hours ago |
15-35596 15 days ago |
15-48077 15 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'] |
chrisflav assignee:chrisflav |
0-57676 16 hours ago |
14-76482 14 days ago |
14-76531 14 days |
27255 |
Louddy author:Louddy |
feat(SkewMonoidAlgebra): 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'] |
chrisflav assignee:chrisflav |
0-57675 16 hours ago |
14-65817 14 days ago |
14-65809 14 days |
27368 |
alreadydone author:alreadydone |
feat(FieldTheory/Finite): minimal polynomial of Frobenius |
for the normal basis theorem at *Formalizing Class Field Theory*
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
37/5 |
Mathlib/Algebra/Algebra/Equiv.lean,Mathlib/Algebra/Algebra/Hom.lean,Mathlib/FieldTheory/Finite/Basic.lean,Mathlib/FieldTheory/Minpoly/Basic.lean |
4 |
6 |
['alreadydone', 'github-actions', 'kckennylau'] |
riccardobrasca assignee:riccardobrasca |
0-57674 16 hours ago |
7-67200 7 days ago |
8-32974 8 days |
27461 |
IvanRenison author:IvanRenison |
feat(Combinatorics/SimpleGraph/Paths): add lemma `SimpleGraph.Walk.IsPath.mem_support_iff_exists_append` |
This contribution was created as part of the Utrecht Summerschool "Formalizing Mathematics in Lean" in July 2025.
---
[](https://gitpod.io/from-referrer/)
|
t-combinatorics |
14/0 |
Mathlib/Combinatorics/SimpleGraph/Paths.lean |
1 |
1 |
['github-actions'] |
awainverse assignee:awainverse |
0-57673 16 hours ago |
7-81517 7 days ago |
7-81562 7 days |
27840 |
CBirkbeck author:CBirkbeck |
feat(NumberTheory/ModularForms/EisensteinSeries): define gammaSetN |
---
[](https://gitpod.io/from-referrer/)
|
t-number-theory |
75/1 |
Mathlib/NumberTheory/ModularForms/EisensteinSeries/Defs.lean |
1 |
1 |
['github-actions'] |
nobody |
0-57145 15 hours ago |
0-57855 16 hours ago |
0-57898 16 hours |
27743 |
alreadydone author:alreadydone |
feat(NumberTheory): Frobenius number exists, ℕ is Noetherian semiring & Sylver coinage |
+ The Frobenius number of a set of natural numbers exist iff the set has gcd 1 and doesn't contain 1.
+ All additive submonoids (= ideals) of ℕ are finitely generated.
+ The game of Sylver coinage always terminates.
This is the outcome of a course project at Heidelberg University: [matematiflo.github.io/CompAssistedMath2025](https://matematiflo.github.io/CompAssistedMath2025/)
Co-authored-by: Daniel Buth @greymatter8
Co-authored-by: Sebastian Meier @SebastianMeierUni
---
FrobeniusNumber is a leaf file so I think doubling its imports is okay.
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebra
t-combinatorics
t-number-theory
label:t-algebra$ |
259/28 |
Mathlib/Data/Set/Finite/Basic.lean,Mathlib/LinearAlgebra/FreeModule/PID.lean,Mathlib/NumberTheory/FrobeniusNumber.lean,Mathlib/RingTheory/Ideal/NatInt.lean,Mathlib/RingTheory/PrincipalIdealDomain.lean |
5 |
2 |
['github-actions', 'vihdzp'] |
nobody |
0-56867 15 hours ago |
1-52465 1 day ago |
1-78067 1 day |
26981 |
JovanGerb author:JovanGerb |
chore: golf using `grw` |
This PR cleans up some proofs using `grw`. It also tags a few lemmas with `@[gcongr]` that were required for the proofs.
---
- [ ] depends on: #26907
[](https://gitpod.io/from-referrer/)
|
large-import |
179/202 |
Archive/Wiedijk100Theorems/CubingACube.lean,Mathlib/Algebra/Category/ModuleCat/Topology/Basic.lean,Mathlib/Algebra/Group/Subgroup/Basic.lean,Mathlib/Algebra/Group/Subgroup/Map.lean,Mathlib/Algebra/Lie/Engel.lean,Mathlib/Algebra/Lie/IdealOperations.lean,Mathlib/Algebra/Module/Submodule/IterateMapComap.lean,Mathlib/Algebra/Order/Archimedean/Basic.lean,Mathlib/Algebra/Order/CauSeq/BigOperators.lean,Mathlib/Algebra/Order/Field/Basic.lean,Mathlib/Algebra/Order/Group/Multiset.lean,Mathlib/Algebra/Order/Kleene.lean,Mathlib/Algebra/Order/Rearrangement.lean,Mathlib/Algebra/Order/Ring/Unbundled/Basic.lean,Mathlib/Analysis/BoxIntegral/Integrability.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Isometric.lean,Mathlib/Analysis/Calculus/ContDiff/Bounds.lean,Mathlib/Analysis/Convex/Gauge.lean,Mathlib/Analysis/Convex/Slope.lean,Mathlib/Analysis/Distribution/SchwartzSpace.lean,Mathlib/Analysis/Normed/Affine/AddTorsor.lean,Mathlib/Analysis/Normed/Order/UpperLower.lean,Mathlib/Analysis/NormedSpace/OperatorNorm/NNNorm.lean,Mathlib/Analysis/Oscillation.lean,Mathlib/Analysis/SpecialFunctions/Pow/NNReal.lean,Mathlib/Combinatorics/Additive/AP/Three/Behrend.lean,Mathlib/Combinatorics/Hall/Finite.lean,Mathlib/Data/NNReal/Defs.lean,Mathlib/Data/Real/Cardinality.lean,Mathlib/Dynamics/Ergodic/MeasurePreserving.lean,Mathlib/FieldTheory/IntermediateField/Adjoin/Basic.lean,Mathlib/LinearAlgebra/AffineSpace/Ordered.lean,Mathlib/MeasureTheory/Covering/LiminfLimsup.lean,Mathlib/MeasureTheory/Integral/Bochner/Basic.lean,Mathlib/MeasureTheory/Integral/Bochner/Set.lean,Mathlib/MeasureTheory/Integral/Bochner/VitaliCaratheodory.lean,Mathlib/MeasureTheory/Integral/DominatedConvergence.lean,Mathlib/MeasureTheory/Integral/IntegralEqImproper.lean,Mathlib/MeasureTheory/Measure/Content.lean,Mathlib/MeasureTheory/Measure/EverywherePos.lean,Mathlib/MeasureTheory/Measure/IntegralCharFun.lean,Mathlib/MeasureTheory/Measure/Lebesgue/Basic.lean,Mathlib/MeasureTheory/Measure/Stieltjes.lean,Mathlib/MeasureTheory/OuterMeasure/Caratheodory.lean,Mathlib/MeasureTheory/OuterMeasure/Induced.lean,Mathlib/MeasureTheory/OuterMeasure/OfFunction.lean,Mathlib/NumberTheory/ClassNumber/AdmissibleCardPowDegree.lean,Mathlib/NumberTheory/FLT/Polynomial.lean,Mathlib/NumberTheory/ModularForms/JacobiTheta/TwoVariable.lean,Mathlib/NumberTheory/Transcendental/Lindemann/AnalyticalPart.lean,Mathlib/Order/Basic.lean,Mathlib/Order/BooleanAlgebra/Basic.lean,Mathlib/Order/Closure.lean,Mathlib/Order/ConditionallyCompleteLattice/Basic.lean,Mathlib/Order/Height.lean,Mathlib/Order/Interval/Set/Monotone.lean,Mathlib/Order/Monotone/Extension.lean,Mathlib/Order/PrimeSeparator.lean,Mathlib/Probability/Martingale/Upcrossing.lean,Mathlib/Probability/Process/HittingTime.lean,Mathlib/RingTheory/Ideal/Operations.lean,Mathlib/RingTheory/MvPowerSeries/PiTopology.lean,Mathlib/RingTheory/Polynomial/Basic.lean,Mathlib/SetTheory/Cardinal/Arithmetic.lean,Mathlib/SetTheory/Cardinal/Ordinal.lean,Mathlib/SetTheory/Ordinal/Basic.lean,Mathlib/SetTheory/Ordinal/Enum.lean,Mathlib/SetTheory/Ordinal/FixedPointApproximants.lean,Mathlib/Topology/Maps/Basic.lean,Mathlib/Topology/MetricSpace/Holder.lean,Mathlib/Topology/MetricSpace/Kuratowski.lean,Mathlib/Topology/MetricSpace/Thickening.lean,Mathlib/Topology/NhdsSet.lean,Mathlib/Topology/Order.lean |
74 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
0-54743 15 hours ago |
1-36724 1 day ago |
1-42159 1 day |
27400 |
dleijnse author:dleijnse |
feat: define geometrically reduced algebras |
Define geometrically reduced algebras, and prove that if all finitely generated subalgebras of an algebra `A` are geometrically reduced, then `A` is geometrically reduced.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-algebra
label:t-algebra$ |
111/0 |
Mathlib.lean,Mathlib/RingTheory/Nilpotent/GeometricallyReduced.lean |
2 |
23 |
['dleijnse', 'github-actions', 'kckennylau'] |
nobody |
0-54567 15 hours ago |
9-46644 9 days ago |
9-46690 9 days |
27839 |
CBirkbeck author:CBirkbeck |
feat(NumberTheory/ModularForms/EisensteinSeries): |
define normalised Eisenstein series in preparation for giving their q-expansions.
---
[](https://gitpod.io/from-referrer/)
|
t-number-theory |
11/0 |
Mathlib/NumberTheory/ModularForms/EisensteinSeries/Basic.lean |
1 |
1 |
['github-actions'] |
nobody |
0-54457 15 hours ago |
0-58327 16 hours ago |
0-58377 16 hours |
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 |
maintainer-merge
t-category-theory
|
169/0 |
Mathlib.lean,Mathlib/CategoryTheory/Functor/Derived/PointwiseRightDerived.lean |
2 |
13 |
['github-actions', 'joelriou', 'robin-carlier'] |
robin-carlier assignee:robin-carlier |
0-53060 14 hours ago |
0-81475 22 hours ago |
45-19423 45 days |
27457 |
grunweg author:grunweg |
feat(LocallyIntegrable): generalise the first half of the file to enorms |
---
This is not exhaustive; all `smul` lemmas can also be generalised (assuming suitable typeclasses).
That will happen in a separate PR.
[](https://gitpod.io/from-referrer/)
|
carleson
maintainer-merge
t-measure-probability
|
90/48 |
Mathlib/MeasureTheory/Function/LocallyIntegrable.lean,Mathlib/MeasureTheory/Integral/IntegrableOn.lean |
2 |
11 |
['YaelDillies', 'github-actions', 'grunweg'] |
EtienneC30 assignee:EtienneC30 |
0-52940 14 hours ago |
0-52940 14 hours ago |
8-4256 8 days |
27846 |
euprunin author:euprunin |
chore(Algebra/Group): golf `range_eq_image_or_of_mulSupport_subset` using `grind` |
|
maintainer-merge
t-algebra
label:t-algebra$ |
1/4 |
Mathlib/Algebra/Group/Support.lean |
1 |
2 |
['github-actions', 'grunweg'] |
nobody |
0-51619 14 hours ago |
0-51619 14 hours ago |
0-53559 14 hours |
27810 |
euprunin author:euprunin |
chore(Algebra/BigOperators): golf `prod_list_map_count` using `grind [Finset.prod_congr]` |
|
maintainer-merge
t-algebra
label:t-algebra$ |
1/5 |
Mathlib/Algebra/BigOperators/Group/Finset/Basic.lean |
1 |
2 |
['github-actions', 'grunweg'] |
nobody |
0-51210 14 hours ago |
0-51210 14 hours ago |
0-82311 22 hours |
27811 |
euprunin author:euprunin |
chore(Algebra/PresentedMonoid): golf `ext` using `grind [Set.eqOn_range]` |
|
maintainer-merge
t-algebra
label:t-algebra$ |
1/4 |
Mathlib/Algebra/PresentedMonoid/Basic.lean |
1 |
2 |
['github-actions', 'grunweg'] |
nobody |
0-51197 14 hours ago |
0-51197 14 hours ago |
0-82227 22 hours |
27808 |
euprunin author:euprunin |
chore(Algebra): golf `surj_of_gcd_domain`, `toCommMonoid_injective`, `f_eq`, `eq_top_of_invtSubmodule_ne_bot` and `dvd_mul_sub_mul_mul_left_of_dvd` using `grind` |
|
maintainer-merge
t-algebra
label:t-algebra$ |
5/13 |
Mathlib/Algebra/GCDMonoid/IntegrallyClosed.lean,Mathlib/Algebra/Group/Ext.lean,Mathlib/Algebra/Homology/Embedding/HomEquiv.lean,Mathlib/Algebra/Lie/Weights/RootSystem.lean,Mathlib/Algebra/Ring/Divisibility/Lemmas.lean |
5 |
2 |
['github-actions', 'grunweg'] |
nobody |
0-51183 14 hours ago |
0-51183 14 hours ago |
0-82553 22 hours |
27663 |
ShreckYe author:ShreckYe |
feat(Analysis/SpecialFunctions/Trigonometric/Basic): add the duals named `cos_eq_zero_iff_sin_eq` for the theorems named `sin_eq_zero_iff_cos_eq` in both real and complex cases |
Similar to #27622. These seem missing for cosine case.
I simplified the proofs adapted from `sin_eq_zero_iff_cos_eq` using `simp` compared to the original way of constructing the remaining goal explictly using `exact`. If needed, I can simplify the proofs of the 2 `sin_eq_zero_iff_cos_eq`s too. |
new-contributor
t-analysis
easy
|
8/0 |
Mathlib/Analysis/SpecialFunctions/Trigonometric/Basic.lean |
1 |
6 |
['ShreckYe', 'github-actions', 'themathqueen'] |
nobody |
0-49997 13 hours ago |
1-78741 1 day ago |
3-23593 3 days |
27699 |
mans0954 author:mans0954 |
refactor(Analysis/Normed/Module/Dual): Abbrev for topological dual |
The concept of a topological dual can be defined whenever `E →L[𝕜] 𝕜` makes sense.
Discussion: https://github.com/leanprover-community/mathlib4/pull/26345/files#r2234132483
---
[](https://gitpod.io/from-referrer/)
|
|
130/124 |
Mathlib/Analysis/InnerProductSpace/Adjoint.lean,Mathlib/Analysis/InnerProductSpace/Dual.lean,Mathlib/Analysis/Normed/Module/Dual.lean,Mathlib/Analysis/Normed/Module/WeakDual.lean,Mathlib/Analysis/VonNeumannAlgebra/Basic.lean,Mathlib/MeasureTheory/Function/AEEqOfIntegral.lean,Mathlib/MeasureTheory/Measure/CharacteristicFunction.lean,Mathlib/MeasureTheory/Measure/IntegralCharFun.lean,Mathlib/Probability/Distributions/Gaussian/Basic.lean,Mathlib/Probability/Moments/CovarianceBilin.lean,Mathlib/Topology/Algebra/Module/LinearMap.lean,docs/overview.yaml,docs/undergrad.yaml |
13 |
21 |
['eric-wieser', 'github-actions', 'j-loreaux', 'mans0954', 'themathqueen'] |
nobody |
0-48013 13 hours ago |
2-42312 2 days ago |
2-44950 2 days |
27845 |
themathqueen author:themathqueen |
feat(Analysis/InnerProductSpace/Adjoint): some API for `innerSL` |
In [bra-ket notation](https://en.wikipedia.org/wiki/Bra–ket_notation), these are:
- $\langle x|^\dagger=|x\rangle$,
- $f\circ|x\rangle=|f(x)\rangle$,
- $\langle x|\circ f=\langle f^\dagger(x)|$,
where $\langle x|$ is `innerSL _ x`, and $|x\rangle$ is `(lsmul _ _).flip x`.
---
[](https://gitpod.io/from-referrer/)
|
t-analysis |
19/0 |
Mathlib/Analysis/InnerProductSpace/Adjoint.lean,Mathlib/Analysis/NormedSpace/OperatorNorm/Mul.lean |
2 |
1 |
['github-actions'] |
nobody |
0-44806 12 hours ago |
0-53644 14 hours ago |
0-53696 14 hours |
27849 |
robin-carlier author:robin-carlier |
feat(CategoryTheory/Bicategory/Functor): strictly unitary lax/pseudo functors |
We define strictly unitary lax/pseudo functors between bicategories. A lax (resp. pseudo-)functor from `C` to `D` is strictly unitary if `F.map(𝟙 X) = 𝟙 (F.obj X)` and if the 2-cell `mapId` is the identity 2-cell induced by this equality. We provide a constructor for those that do not require the `mapId` field.
Although this structure is somewhat "evil" from a purely categorical perspective (it mentions non-definitonal equality of objects in a 1-category), these class of functors are of interest: strictly unitary lax functors are part of the definition of the Duskin nerve of a bicategory (which embeds bicategories in the theory of simplicial sets), while strictly unitary pseudofunctors are part of the definition of the 2-nerve of a bicategory, which embeds bicategories into the theory of simplicial categories.
This PR is part of an ongoing work that will hopefully culminate with the construction of the Duskin Nerve, as well as a proof of the fact that the Duskin nerve of a locally groupoidal bicategory is a quasicategory.
---
Two designs were possible here: making `StrictlyUnitary` a class on lax/pseudo-functors to state that some functors/constructions are strictly unitary, or bundling it as a structure on its own.
Since my plan for the following is to use the type of strictly lax unitary functors between some bicategories (e.g to define lax-composable arrows in a bicategory `C`, which will be by definition `StrictlyUnitaryLaxFunctor (LocallyDiscrete (Fin n)) C`), I chose to bundle them directly, to avoid an extra layer when working with the type of those objects.
I did include strict associativity for strictly unitary lax functors but not for pseudofunctors. The reason is that the Duskin nerve mentions the 1-category of bicategories and strictly unitary lax functors (hence, this strict associativity/unitality), but the 2-nerve mentions the bicategory of bicategories, strictly unitary pseudofunctors and "icons" (identity-component oplax natural transformations): the statement for associativity for pseudofunctors will wait for icons, and will probably not be stated as an equality of pseudofunctors.
[](https://gitpod.io/from-referrer/)
|
t-category-theory |
318/0 |
Mathlib.lean,Mathlib/CategoryTheory/Bicategory/Functor/StrictlyUnitary.lean |
2 |
1 |
['github-actions'] |
nobody |
0-44795 12 hours ago |
0-45007 12 hours ago |
0-45060 12 hours |
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-algebraic-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 |
6 |
['github-actions', 'grunweg', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'robin-carlier'] |
nobody |
0-42888 11 hours ago |
1-75147 1 day ago |
47-42176 47 days |
27835 |
edegeltje author:edegeltje |
feat(Tactic): ring modulo a given characteristic (resurrection of #10765, attempt two) |
This used to be #10765 by Anne Baanen before the great forkening.
> This PR extends the `ring` tactic with a new config argument `char` which will try to reduce all constant terms modulo the given characteristic. This allows `ring` to prove e.g. `(x + y)^3 = x^3 + y^3` in characteristic 3. This is a simpler and faster way to do so than what we had before: `repeat { ring; reduce_mod_char }` becomes `ring (config := { char := 3 })`.
>
> The first step is to split off the required `CharP` definitions, since `Mathlib.Algebra.CharP.Basic` already requires the `ring` tactic.
>
> To perform the reduction modulo the given characteristic, I implemented `reduceCast` which reduces a raw integer, and wrapped it in `reduceResult` that takes a `NormNum.Result` for easy use. We need to pass through quite a few parameters into `reduceResult` so maybe it's worth defining a structure, or reusing `Cache` for this.
>
> Then it's basically a case of replacing every place where `ring` constructs a numeral with a call to `reduceResult`.
>
> Limitations:
>
> * `ring` doesn't attempt to detect the characteristic by itself, you need to pass it in explicitly. Trying to infer a `CharP` instance at each point sounds quite expensive.
>
> * Since the support for `%` in `NormNum` only exists for integers, I implemented the reduction only when a `Ring` instance is available. It is still sound in the semiring case, just not complete.
>
> * We could optimize exponentiation in the specific case where the characteristic `p` is a prime that divides the exponent `n`: `(x + y)^n = x^n + y^n`. I'll leave that to future work.
>
---
[](https://gitpod.io/from-referrer/)
|
migrated-from-branch
large-import
t-meta
|
309/134 |
Mathlib/LinearAlgebra/Eigenspace/Basic.lean,Mathlib/RingTheory/MvPolynomial/Basic.lean,Mathlib/Tactic/LinearCombination.lean,Mathlib/Tactic/Module.lean,Mathlib/Tactic/Polyrith.lean,Mathlib/Tactic/Ring/Basic.lean,Mathlib/Tactic/Ring/Compare.lean,Mathlib/Tactic/Ring/RingNF.lean,MathlibTest/ring_compare.lean,MathlibTest/ring_mod_char.lean |
10 |
2 |
['edegeltje', 'github-actions'] |
joneugster assignee:joneugster |
0-42137 11 hours ago |
0-42344 11 hours ago |
0-42356 11 hours |
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
---
[](https://gitpod.io/from-referrer/) |
t-algebra label:t-algebra$ |
35/0 |
Mathlib/Algebra/QuadraticDiscriminant.lean |
1 |
4 |
['github-actions', 'tb65536', 'upobir'] |
chrisflav assignee:chrisflav |
0-41515 11 hours ago |
43-67304 1 month ago |
43-67348 43 days |
27847 |
euprunin author:euprunin |
chore(Algebra): avoid duplicating proofs by reusing existing theorems or lemmas |
|
t-algebra label:t-algebra$ |
9/36 |
Mathlib/Algebra/Homology/Embedding/Extend.lean,Mathlib/Algebra/MvPolynomial/Rename.lean,Mathlib/Algebra/Order/Group/Abs.lean,Mathlib/Algebra/Order/Ring/Unbundled/Rat.lean,Mathlib/Algebra/Polynomial/Degree/Lemmas.lean,Mathlib/Algebra/Polynomial/Monic.lean |
6 |
6 |
['github-actions', 'grunweg', 'kbuzzard'] |
nobody |
0-40851 11 hours ago |
0-52503 14 hours ago |
0-52556 14 hours |
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 |
8 |
['YaelDillies', 'agjftucker', 'github-actions', 'igorkhavkine', 'mathlib4-dependent-issues-bot'] |
sgouezel assignee:sgouezel |
0-39945 11 hours ago |
37-2400 1 month ago |
37-74538 37 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 |
2 |
['JovanGerb', 'github-actions'] |
nobody |
0-38814 10 hours ago |
26-42271 26 days ago |
26-42326 26 days |
27451 |
kckennylau author:kckennylau |
feat(RingTheory/Valuation): define ball, closed ball, and sphere |
*From the 2025 Local Class Field Theory Workshop.*
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
27/0 |
Mathlib/RingTheory/Valuation/Basic.lean |
1 |
8 |
['JovanGerb', 'github-actions', 'pechersky', 'wwylele'] |
nobody |
0-38610 10 hours ago |
8-30380 8 days ago |
8-30429 8 days |
27852 |
raja-19 author:raja-19 |
feat(Order): add Teichmuller-Tukey lemma |
We define the notion of being of finite character for a family of sets and prove the Teichmuller-Tukey lemma.
This contribution was created as part of the Utrecht Summerschool "Formalizing Mathematics in Lean" in July 2025.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-order
|
61/0 |
Mathlib.lean,Mathlib/Order/TeichmullerTukey.lean |
2 |
1 |
['github-actions'] |
nobody |
0-37907 10 hours ago |
0-37916 10 hours ago |
0-37963 10 hours |
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$ |
52/26 |
Mathlib/Analysis/Fourier/AddCircleMulti.lean,Mathlib/Analysis/RCLike/Lemmas.lean,Mathlib/Topology/Algebra/Module/FiniteDimension.lean,Mathlib/Topology/Algebra/Module/ModuleTopology.lean |
4 |
12 |
['erdOne', 'github-actions', 'leanprover-bot', 'matthewjasper', 'ocfnash', 'riccardobrasca'] |
ocfnash assignee:ocfnash |
0-37124 10 hours ago |
90-76038 2 months ago |
92-44334 92 days |
27570 |
bryangingechen author:bryangingechen |
fix: do not remove reactions if the corresponding label is still present on the PR |
Recently the reaction bot on Zulip has been observed to add a reaction and then remove it shortly afterwards (mainly the reactions corresponding to the `ready-to-merge` and `delegated` labels). The mechanism seems to be the following:
- a maintainer writes a comment like "bors merge" (or "bors d+") on a PR that has been `maintainer-merge`'d
- `zulip_emoji_merge_delegate.yaml` and `zulip_emoji_merge_delegate_wf.yaml` react to this comment and:
- simultaneously adds the "ready-to-merge" and removes the `maintainer-merge` label
- adds the "merge" emoji reaction on Zulip
- the `zulip_emoji_labelling.yaml` workflow reacts to the `maintainer-merge` label being removed, and clears the "merge" emoji as well. See [this log](https://github.com/leanprover-community/mathlib4/actions/runs/16270158496/job/45935446666#step:5:30) (which removes the "delegated" emoji).
We change the `zulip_emoji_labelling.yaml` workflow so that it passes the current list of labels on the PR to the `zulip_emoji_reactions.py` script, and also change the script so that it only removes a reaction if the corresponding label is NOT present.
cf. https://leanprover.zulipchat.com/#narrow/channel/345428-mathlib-reviewers/topic/merge.2Fdelegate.20emojis.20bot/near/528289834
---
[](https://gitpod.io/from-referrer/)
|
maintainer-merge
CI
|
47/18 |
.github/workflows/zulip_emoji_labelling.yaml,scripts/zulip_emoji_reactions.py |
2 |
16 |
['adomani', 'bryangingechen', 'github-actions', 'grunweg'] |
nobody |
0-35932 9 hours ago |
0-35998 9 hours ago |
5-2781 5 days |
27795 |
xroblot author:xroblot |
chore(RingTheory/Localization/AtPrime): move file to `RingTheory/Localization/AtPrime/Basic.lean` |
Create the directory `Mathlib/RingTheory/Localization/AtPrime` and move the file `Mathlib/RingTheory/Localization/AtPrime.lean` to `Mathlib/RingTheory/Localization/AtPrime/Basic.lean`.
This is needed to make way for the new file `Mathlib/RingTheory/Localization/AtPrime/Extension.lean` in #27706 since the results of this file cannot be added to the file `Mathlib/RingTheory/Localization/AtPrime.lean` because of circular dependencies.
The deprecated module is added in the following PR: #27796
---
[](https://gitpod.io/from-referrer/)
|
file-removed
maintainer-merge
easy
|
12/12 |
Mathlib.lean,Mathlib/AlgebraicGeometry/StructureSheaf.lean,Mathlib/RingTheory/GradedAlgebra/HomogeneousLocalization.lean,Mathlib/RingTheory/Ideal/AssociatedPrime/Localization.lean,Mathlib/RingTheory/Ideal/GoingUp.lean,Mathlib/RingTheory/Ideal/MinimalPrime/Localization.lean,Mathlib/RingTheory/LocalProperties/Basic.lean,Mathlib/RingTheory/LocalProperties/Submodule.lean,Mathlib/RingTheory/LocalRing/LocalSubring.lean,Mathlib/RingTheory/LocalRing/ResidueField/Ideal.lean,Mathlib/RingTheory/Localization/AtPrime/Basic.lean,Mathlib/RingTheory/Localization/LocalizationLocalization.lean,Mathlib/RingTheory/SurjectiveOnStalks.lean |
13 |
3 |
['github-actions', 'grunweg', 'mathlib4-merge-conflict-bot'] |
nobody |
0-35733 9 hours ago |
0-35755 9 hours ago |
0-83394 23 hours |
27853 |
JovanGerb author:JovanGerb |
chore(Data/Int/Interval): use `omega` |
---
[](https://gitpod.io/from-referrer/)
|
t-data
maintainer-merge
|
20/32 |
Mathlib/Data/Int/Interval.lean |
1 |
4 |
['JovanGerb', 'euprunin', 'github-actions', 'grunweg'] |
nobody |
0-35701 9 hours ago |
0-35701 9 hours ago |
0-37254 10 hours |
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 |
0-33918 9 hours ago |
27-60350 27 days ago |
30-6149 30 days |
27040 |
Scarlett-le author:Scarlett-le |
feat(Geometry/Euclidean/Sphere/Power): add power of a point theorems |
Add the definition of power of a point and fundamental theorems relating
point positions to intersection distances:
* `Sphere.power`: The power of a point with respect to a sphere, defined as
the square of the distance from the point to the center minus the square
of the radius.
* `Sphere.power_eq_zero_iff_mem_sphere`: A point lies on the sphere if and
only if its power is zero.
* `Sphere.power_pos_iff_dist_center_gt_radius`: The power is positive if and
only if the point is outside the sphere.
* `Sphere.power_neg_iff_dist_center_lt_radius`: The power is negative if and
only if the point is inside the sphere.
* `Sphere.mul_dist_eq_power_of_dist_center_gt_radius`: For external points,
the product of intersection distances equals the power.
* `Sphere.mul_dist_eq_neg_power_of_dist_center_lt_radius`: For internal points,
the product equals the negative power.
* `Sphere.mul_dist_eq_abs_power`: General form relating intersection distance
products to absolute power.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-euclidean-geometry
|
138/1 |
Mathlib/Geometry/Euclidean/Sphere/Power.lean |
1 |
4 |
['alreadydone', 'github-actions', 'jsm28'] |
jsm28 assignee:jsm28 |
0-33070 9 hours ago |
20-50293 20 days ago |
20-50833 20 days |
27378 |
peakpoint author:peakpoint |
refactor(Geometry/Euclidean/Projection): redefine projection and reflection for affine subspaces |
This PR continues the work from #25578.
Original PR: https://github.com/leanprover-community/mathlib4/pull/25578 |
new-contributor
t-euclidean-geometry
|
316/317 |
Mathlib/Analysis/Normed/Affine/ContinuousAffineMap.lean,Mathlib/Analysis/Normed/Affine/Isometry.lean,Mathlib/Geometry/Euclidean/Circumcenter.lean,Mathlib/Geometry/Euclidean/Projection.lean |
4 |
6 |
['github-actions', 'jsm28', 'leanprover-community-bot-assistant', 'peakpoint'] |
nobody |
0-32701 9 hours ago |
5-32605 5 days ago |
9-1941 9 days |
27857 |
euprunin author:euprunin |
chore(Analysis/SpecialFunctions): golf entire `rpow_eq_top_of_nonneg` using `simp` |
|
maintainer-merge
t-analysis
|
1/6 |
Mathlib/Analysis/SpecialFunctions/Pow/NNReal.lean |
1 |
2 |
['eric-wieser', 'github-actions', 'grunweg'] |
nobody |
0-32139 8 hours ago |
0-35353 9 hours ago |
0-35860 9 hours |
26726 |
euprunin author:euprunin |
chore: golf Algebra/ using `grind` |
|
maintainer-merge
t-algebra
label:t-algebra$ |
40/169 |
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/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/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,Mathlib/AlgebraicTopology/DoldKan/Homotopies.lean |
25 |
25 |
['euprunin', 'github-actions', 'grunweg', 'leanprover-bot', 'leanprover-community-bot-assistant', 'leanprover-community-mathlib4-bot'] |
nobody |
0-31961 8 hours ago |
1-73947 1 day ago |
28-80364 28 days |
27856 |
euprunin author:euprunin |
chore(RingTheory/PowerSeries): golf entire `trunc_one` using `grind` |
|
maintainer-merge
t-algebra
label:t-algebra$ |
1/6 |
Mathlib/RingTheory/PowerSeries/Trunc.lean |
1 |
3 |
['eric-wieser', 'euprunin', 'github-actions', 'grunweg'] |
nobody |
0-31038 8 hours ago |
0-35715 9 hours ago |
0-36233 10 hours |
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'] |
dagurtomas assignee:dagurtomas |
0-27993 7 hours ago |
39-20036 1 month ago |
39-21327 39 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'] |
mariainesdff assignee:mariainesdff |
0-27993 7 hours ago |
82-32372 2 months ago |
148-32355 148 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'] |
bryangingechen assignee:bryangingechen |
0-27992 7 hours ago |
31-35732 1 month ago |
50-86317 50 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'] |
b-mehta assignee:b-mehta |
0-27991 7 hours ago |
50-86166 1 month ago |
50-86149 50 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'] |
awainverse assignee:awainverse |
0-27991 7 hours ago |
49-68743 1 month ago |
49-68727 49 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'] |
jcommelin assignee:jcommelin |
0-27990 7 hours ago |
41-50677 1 month ago |
41-50739 41 days |
26398 |
ChrisHughes24 author:ChrisHughes24 |
feat(ModelTheory): definable functions |
---
Possibly this should be generalized to partial functions.
I migrated the PR by hand instead of using the script.
- [x] depends on: #20166
- [x] depends on: #20161
- [x] depends on: #20115
- [x] depends on: #20174
- [x] depends on: #20175
- [x] depends on: #21948
[](https://gitpod.io/from-referrer/)
|
t-logic |
618/0 |
Mathlib.lean,Mathlib/ModelTheory/FunctionalFormula.lean |
2 |
3 |
['ChrisHughes24', 'github-actions', 'mathlib4-dependent-issues-bot'] |
fpvandoorn assignee:fpvandoorn |
0-27989 7 hours ago |
37-85257 1 month ago |
37-85516 37 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'] |
joelriou assignee:joelriou |
0-27988 7 hours ago |
36-19923 1 month ago |
36-20048 36 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$ |
205/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'] |
kbuzzard assignee:kbuzzard |
0-27987 7 hours ago |
27-74043 27 days ago |
27-74072 27 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'] |
PatrickMassot assignee:PatrickMassot |
0-27986 7 hours ago |
15-69770 15 days ago |
15-69931 15 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'] |
alreadydone assignee:alreadydone |
0-27985 7 hours ago |
18-77100 18 days ago |
19-41607 19 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'] |
mattrobball assignee:mattrobball |
0-27983 7 hours ago |
16-78929 16 days ago |
16-79828 16 days |
27424 |
vihdzp author:vihdzp |
feat: interval in archimedean field contains fraction with large enough denominator |
This is a slight generalization of `exists_rat_btwn` that can be used, for instance, to prove that there's a dyadic rational between any two elements.
---
[](https://gitpod.io/from-referrer/)
|
maintainer-merge
t-algebra
label:t-algebra$ |
13/11 |
Mathlib/Algebra/Order/Archimedean/Basic.lean |
1 |
2 |
['Ruben-VandeVelde', 'github-actions'] |
mattrobball assignee:mattrobball |
0-27982 7 hours ago |
8-48012 8 days ago |
8-81175 8 days |
27472 |
guelmi94 author:guelmi94 |
feat(Combinatorics/SimpleGraph/Walk): add lemma `support_injective` |
This contribution was created as part of the Utrecht Summerschool "Formalizing Mathematics in Lean" in July 2025.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-combinatorics
|
3/0 |
Mathlib/Combinatorics/SimpleGraph/Walk.lean |
1 |
1 |
['github-actions'] |
b-mehta assignee:b-mehta |
0-27982 7 hours ago |
7-65386 7 days ago |
7-65435 7 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/)
|
maintainer-merge
t-euclidean-geometry
|
86/0 |
Mathlib/Analysis/Convex/Between.lean |
1 |
3 |
['github-actions', 'jsm28'] |
jsm28 assignee:jsm28 |
0-26113 7 hours ago |
0-26113 7 hours ago |
32-54403 32 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* |
maintainer-merge
t-algebra
label:t-algebra$ |
76/3 |
Mathlib/Algebra/Module/ZLattice/Basic.lean,Mathlib/Algebra/Module/ZLattice/Covolume.lean,Mathlib/GroupTheory/Index.lean,Mathlib/LinearAlgebra/Determinant.lean |
4 |
13 |
['github-actions', 'leanprover-community-bot-assistant', 'madvorak', 'mathlib4-dependent-issues-bot', 'tb65536', 'xroblot'] |
nobody |
0-23595 6 hours ago |
0-29770 8 hours ago |
50-56463 50 days |
27864 |
BoltonBailey author:BoltonBailey |
feat(Data/{Finset,Multiset}/Sort): give sort functions ≤ default argument |
Changes the `Finset.sort` and `Multiset.sort` functions to take `≤` as the default relation argument. Then removes this argument where possible through the rest of the library.
This involves switching the order of arguments, but I think this is fine, as this function is mostly called by dot notation anyway, and I think it is more typical for the first argument of such functions to have the type that matches the namespace.
Thanks to @eric-wieser for suggesting this approach
---
[](https://gitpod.io/from-referrer/)
|
|
121/97 |
Mathlib/Algebra/Polynomial/Basic.lean,Mathlib/Data/Finset/Sort.lean,Mathlib/Data/Multiset/Sort.lean,Mathlib/Data/Nat/Nth.lean,Mathlib/GroupTheory/Perm/Cycle/Factors.lean,Mathlib/GroupTheory/Perm/Sign.lean,Mathlib/Logic/Equiv/Finset.lean,Mathlib/Logic/Equiv/Multiset.lean,Mathlib/NumberTheory/ADEInequality.lean |
9 |
4 |
['BoltonBailey', 'eric-wieser', 'github-actions'] |
nobody |
0-20618 5 hours ago |
0-29589 8 hours ago |
0-29852 8 hours |
27159 |
Parcly-Taxel author:Parcly-Taxel |
feat: IMO 1997 Q3 |
|
IMO |
114/0 |
Archive.lean,Archive/Imo/Imo1997Q3.lean |
2 |
9 |
['Parcly-Taxel', 'eric-wieser', 'github-actions', 'jsm28'] |
jsm28 assignee:jsm28 |
0-18263 5 hours ago |
17-70152 17 days ago |
17-70140 17 days |
27866 |
xroblot author:xroblot |
feat(Algebra/IsScalarTower): add transitivity results |
Add the following:
Let `R ⊆ S ⊆ T ⊆ U` be a tower of rings. If `R ⊆ S ⊆ T`, `R ⊆ T ⊆ U` and `S ⊆ T ⊆ U` are scalar towers, then `R ⊆ S ⊆ U` is also a scalar tower.
Add also, the "right side" version where we deduce that `R ⊆ T ⊆ U` is a scalar tower.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
22/0 |
Mathlib/Algebra/Algebra/Tower.lean |
1 |
1 |
['github-actions'] |
nobody |
0-17551 4 hours ago |
0-17622 4 hours ago |
0-17656 4 hours |
27855 |
eric-wieser author:eric-wieser |
refactor: group matrix norm instance behind scopes |
It's possible that type synonyms are worth exploring here, but this is strictly better than the status quo where it can be easy to forget one of this family of instances.
---
[](https://gitpod.io/from-referrer/)
|
t-analysis |
54/38 |
Mathlib/Analysis/CStarAlgebra/CStarMatrix.lean,Mathlib/Analysis/CStarAlgebra/Matrix.lean,Mathlib/Analysis/Matrix.lean,Mathlib/Analysis/Normed/Algebra/MatrixExponential.lean |
4 |
9 |
['b-mehta', 'eric-wieser', 'github-actions', 'j-loreaux'] |
nobody |
0-12819 3 hours ago |
0-37074 10 hours ago |
0-37119 10 hours |
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/347 |
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/Choose/Central.lean,Mathlib/Data/Nat/Choose/Sum.lean,Mathlib/Data/Nat/Digits/Defs.lean,Mathlib/Data/Real/GoldenRatio.lean,Mathlib/Data/Real/Pi/Bounds.lean,Mathlib/Data/Real/Pi/Irrational.lean,Mathlib/Data/Real/Sign.lean,Mathlib/FieldTheory/Finite/Basic.lean,Mathlib/Geometry/Euclidean/Angle/Unoriented/RightAngle.lean |
168 |
20 |
['Ruben-VandeVelde', 'YaelDillies', 'adomani', 'b-mehta', 'euprunin', 'github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'leanprover-community-mathlib4-bot'] |
nobody |
0-11044 3 hours ago |
0-11044 3 hours ago |
31-41216 31 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$ |
200/3 |
Mathlib.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/Support.lean |
7 |
n/a |
['Thmoas-Guan', 'chrisflav', 'github-actions', 'leanprover-community-bot-assistant', 'mbkybky'] |
nobody |
0-3315 55 minutes ago |
unknown |
unknown |
27107 |
AntoineChambert-Loir author:AntoineChambert-Loir |
feat(GroupTheory/GroupAction/SubMulAction/Combination) : combinations and group actions |
`Nat.Combination X n` is the type all `s : Finset X` such that `s.card = n`.
This PR provides some API for this subtype and the `SubMulAction` it inherits when a group acts on `X`.
It will be used in conjunction with the description of some maximal subgroups of `Equiv.Perm X` to construct primitive actions.
Question on the names: when `X` is a fintype, there is `Finset.powersetCard` that gives the same object, as a `Finset`. But the present PR also applies when `X` is infinite. Then maybe `Nat.Combination` should be renamed as `Set.powersetCard`?
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
318/0 |
Mathlib.lean,Mathlib/Data/Nat/Choose/Basic.lean,Mathlib/GroupTheory/GroupAction/SubMulAction/Combination.lean |
3 |
2 |
['github-actions', 'tb65536'] |
alreadydone assignee:alreadydone |
0-3073 51 minutes ago |
19-26130 19 days ago |
19-26174 19 days |
27865 |
zcyemi author:zcyemi |
feat(Algebra/AddTorsor/Basic) vadd_vsub_vadd |
Add `vadd_vsub_vadd `
```lean
theorem vadd_vsub_vadd (v₁ v₂ : G) (p₁ p₂ : P) : (v₁ +ᵥ p₁) -ᵥ (v₂ +ᵥ p₂) = (v₁ - v₂)
+ (p₁ -ᵥ p₂) := by
rw [vsub_vadd_eq_vsub_sub, vadd_vsub_assoc, add_sub_assoc, ← add_comm_sub]
```
---
[](https://gitpod.io/from-referrer/)
|
maintainer-merge
t-algebra
label:t-algebra$ |
4/0 |
Mathlib/Algebra/AddTorsor/Basic.lean |
1 |
3 |
['github-actions', 'grunweg'] |
nobody |
0-2600 43 minutes ago |
0-2600 43 minutes ago |
0-19573 5 hours |
27860 |
euprunin author:euprunin |
chore(GroupTheory/Coxeter): golf `getElem_alternatingWord` using `grind […]` |
|
t-algebra label:t-algebra$ |
2/26 |
Mathlib/GroupTheory/Coxeter/Basic.lean |
1 |
4 |
['github-actions', 'grunweg'] |
nobody |
0-2104 35 minutes ago |
0-33815 9 hours ago |
0-33859 9 hours |
27859 |
euprunin author:euprunin |
chore(GroupTheory/Coxeter): golf entire `getElem_alternatingWord_swapIndices` using `grind [CoxeterSystem.getElem_alternatingWord]` |
|
t-algebra label:t-algebra$ |
2/8 |
Mathlib/GroupTheory/Coxeter/Basic.lean |
1 |
2 |
['github-actions', 'grunweg'] |
nobody |
0-1870 31 minutes ago |
0-34043 9 hours ago |
0-34093 9 hours |