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 |
24218 |
alreadydone author:alreadydone |
chore(Algebra): remove `mid_assoc` from `IsMulCentral` |
as it is a consequence of left and right associativity in the presence of commutativity. Also change the commutativity condition to use `Commute`.
---
Even without commutativity, left and right associativity of an element `e` in a magma is sufficient to prove that elements of the form `e * x * e` (the "corner" of `e`) form a submagma.
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
31/69 |
Mathlib/Algebra/Algebra/NonUnitalSubalgebra.lean,Mathlib/Algebra/Group/Center.lean,Mathlib/Algebra/GroupWithZero/Center.lean,Mathlib/Algebra/Ring/Center.lean,Mathlib/Algebra/Ring/CentroidHom.lean,Mathlib/Algebra/Star/Center.lean,Mathlib/Algebra/Star/CentroidHom.lean,Mathlib/GroupTheory/Submonoid/Center.lean,Mathlib/LinearAlgebra/Basis/Submodule.lean,Mathlib/LinearAlgebra/QuadraticForm/Basic.lean,Mathlib/RingTheory/Idempotents.lean,Mathlib/RingTheory/NonUnitalSubsemiring/Basic.lean |
12 |
8 |
['alreadydone', 'github-actions', 'mans0954'] |
nobody |
71-42283 2 months ago |
71-57343 2 months ago |
71-57332 71 days |
24405 |
mcdoll author:mcdoll |
refactor(Topology/Algebra/Module/WeakDual): Clean up |
- Move `Dual` and `dualPairing` lower in the import-hierachy
- deduplicate `dualPairing`
- Make `WeakDual` and `WeakSpace` reducible
---
New version of #11500
[](https://gitpod.io/from-referrer/)
|
large-import
t-topology
|
146/162 |
Mathlib.lean,Mathlib/Analysis/Fourier/RiemannLebesgueLemma.lean,Mathlib/Analysis/InnerProductSpace/Adjoint.lean,Mathlib/Analysis/InnerProductSpace/Dual.lean,Mathlib/Analysis/LocallyConvex/WeakSpace.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/FiniteMeasure.lean,Mathlib/Topology/Algebra/Module/Dual.lean,Mathlib/Topology/Algebra/Module/WeakDual.lean,docs/overview.yaml,docs/undergrad.yaml |
14 |
1 |
['github-actions'] |
nobody |
64-9555 2 months ago |
64-18248 2 months ago |
64-18230 64 days |
20719 |
gio256 author:gio256 |
feat(AlgebraicTopology): delaborators for truncated simplicial notations |
We add delaborators for the following notations, introduced in #20688:
- `⦋m⦌ₙ`, which denotes the `m`-dimensional simplex in the `n`-truncated simplex category.
- `X _⦋m⦌ₙ`, which denotes the `m`-th term of an `n`-truncated simplicial object `X`.
- `X ^⦋m⦌ₙ`, which denotes the `m`-th term of an `n`-truncated cosimplicial object `X`.
If `pp.proofs` is set to `true`, we also pretty-print the proof `p : m ≤ n` for all three notations as `⦋m, p⦌ₙ`, `X _⦋m, p⦌ₙ`, and `X ^⦋m, p⦌ₙ`, respectively.
Credit to @kmill for one piece of code and much metaprogramming inspiration.
---
- [x] depends on: #20688
- [x] depends on: #23018
[](https://gitpod.io/from-referrer/)
|
infinity-cosmos
t-category-theory
t-meta
|
525/33 |
Mathlib.lean,Mathlib/AlgebraicTopology/SimplexCategory/Basic.lean,Mathlib/AlgebraicTopology/SimplexCategory/Defs.lean,Mathlib/AlgebraicTopology/SimplicialObject/Basic.lean,Mathlib/Tactic.lean,Mathlib/Tactic/SimplexCategory.lean,Mathlib/Util/Superscript.lean,MathlibTest/SimplexCategory.lean,MathlibTest/SimplicialObject.lean,MathlibTest/superscript.lean,scripts/noshake.json |
11 |
22 |
['eric-wieser', 'gio256', 'github-actions', 'kim-em', 'mathlib4-dependent-issues-bot'] |
eric-wieser assignee:eric-wieser |
60-37292 1 month ago |
60-39933 1 month ago |
69-25073 69 days |
24266 |
plp127 author:plp127 |
feat(Order): `NoBotOrder α` implies `NoMinOrder α` under `IsDirected α (· ≥ ·)` |
Proves that `NoBotOrder α` implies `NoMinOrder α` under `IsDirected α (· ≥ ·)`, and also the dual theorem.
---
[](https://gitpod.io/from-referrer/)
|
t-order |
14/0 |
Mathlib/Order/Directed.lean |
1 |
4 |
['github-actions', 'plp127', 'urkud'] |
nobody |
59-6775 1 month ago |
70-18156 2 months ago |
70-18139 70 days |
23498 |
Ruben-VandeVelde author:Ruben-VandeVelde |
chore(Topology.MetricSpace.Lipschitz): stop depending on Topology.Algebra |
Noticed while playing with the new `directoryDependency` linter. Not sure if these could be proved without assuming the continuity of real multiplication.
Copyright from https://github.com/leanprover-community/mathlib3/pull/1921 and https://github.com/leanprover-community/mathlib4/pull/11840.
---
[](https://gitpod.io/from-referrer/)
|
t-topology |
60/34 |
Mathlib.lean,Mathlib/Analysis/Normed/Group/AddTorsor.lean,Mathlib/Analysis/NormedSpace/Multilinear/Basic.lean,Mathlib/Analysis/SpecialFunctions/Exp.lean,Mathlib/Topology/Algebra/MetricSpace/Lipschitz.lean,Mathlib/Topology/MetricSpace/Algebra.lean,Mathlib/Topology/MetricSpace/IsometricSMul.lean,Mathlib/Topology/MetricSpace/Lipschitz.lean,Mathlib/Topology/MetricSpace/PiNat.lean |
9 |
1 |
['github-actions'] |
nobody |
58-76312 1 month ago |
58-76312 1 month ago |
91-56034 91 days |
24527 |
matthewjasper author:matthewjasper |
feat(Topology/Algebra/Module): Add more theorems for IsModuleTopology |
Add theorems that surjective linear maps to the module topology are open.
Add IsModuleTopology instance for quotients.
Add IsModuleTopology instance for finite dimensional T2 vector spaces over a complete normed field and use it to shorten some proofs.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-algebra
t-topology
label:t-algebra$ |
48/24 |
Mathlib/Topology/Algebra/Module/FiniteDimension.lean,Mathlib/Topology/Algebra/Module/ModuleTopology.lean |
2 |
5 |
['erdOne', 'github-actions', 'matthewjasper'] |
nobody |
58-43435 1 month ago |
58-60505 1 month ago |
60-28803 60 days |
22231 |
pechersky author:pechersky |
feat(Algebra/Valued): `AdicExpansion` initial defns |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-topology
label:t-algebra$ |
299/0 |
Mathlib.lean,Mathlib/Topology/Algebra/Valued/AdicExpansion.lean |
2 |
2 |
['Thmoas-Guan', 'github-actions'] |
nobody |
58-3534 1 month ago |
127-5176 4 months ago |
127-5300 127 days |
22464 |
adomani author:adomani |
feat(CI): declarations diff in Lean |
Rewrites the `declaration_diff` script in Lean.
You can see the effect of the new script in the testing branch #22497.
The new CI step runs in approximately 5mins, but is separate from the `build` step.
---
[](https://gitpod.io/from-referrer/)
|
CI |
151/0 |
.github/workflows/PR_summary_lean.yml,scripts/README.md,scripts/declarations_diff.lean,scripts/declarations_diff_lean_shell_glue.sh |
4 |
6 |
['bryangingechen', 'github-actions', 'grunweg'] |
robertylewis assignee:robertylewis |
53-76872 1 month ago |
118-41117 3 months ago |
118-41105 118 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 |
53-56344 1 month ago |
74-28788 2 months ago |
84-77604 84 days |
22196 |
xyzw12345 author:xyzw12345 |
feat: `lie_ring` tactic and `LieReduce` command |
In this PR, we implement a new tactic that reduces expressions in a `LieRing` to a normal form and checks whether they are equal, and a command which reduces the expression and displays the normal form.
The implementation of this tactic imitates the `ring` tactic, using the `Qq` package to implement a specific reduction algorithm, following the theory of Hall sets and Lyndon words. A reference for the algorithm can be found at, for example, [here](https://personal.math.ubc.ca/~cass/research/pdf/Free.pdf).
This project is the result of a workshop at Peking University, and @siddhartha-gadgil has helped us a lot on understanding the concepts in metaprogramming.
Edit: The changes are reverted to a point where only `AtomM` is used.
Co-authored-by:
@Thmoas-Guan <2300010733@stu.pku.edu.cn>
@yhtq <2100012990@stu.pku.edu.cn>
@Blackfeather007 <2100017455@stu.pku.edu.cn>
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-meta
|
816/2 |
Mathlib.lean,Mathlib/Algebra/Lie/Derivation/AdjointAction.lean,Mathlib/Tactic.lean,Mathlib/Tactic/LieAlgebra/Basic.lean,Mathlib/Tactic/LieAlgebra/LieRingNF.lean,Mathlib/Util/AtomM.lean,MathlibTest/lie_ring.lean,scripts/noshake.json |
8 |
16 |
['bryangingechen', 'eric-wieser', 'faenuccio', 'github-actions', 'grunweg', 'ocfnash', 'siddhartha-gadgil', 'xyzw12345'] |
robertylewis assignee:robertylewis |
52-60207 1 month ago |
128-5306 4 months ago |
128-5296 128 days |
24036 |
Louddy author:Louddy |
feat: add `HeightOneSpectrum.ofPrime` |
Add a definition relating elements of type `HeightOneSpectrum R` with the (nonzero) prime elements of the monoid with zero `Ideal R`. (Note the distinction between `Prime` and `Ideal.IsPrime`).
The documentation string is inspired from [Ideal.prime_iff_isPrime](https://leanprover-community.github.io/mathlib4_docs/Mathlib/RingTheory/DedekindDomain/Ideal.html#Ideal.prime_iff_isPrime).
This was discussed [#mathlib4 > Placing a definition in `DedekindDomain.Ideal` @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Placing.20a.20definition.20in.20.60DedekindDomain.2EIdeal.60/near/511647129).
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-algebra
label:t-algebra$ |
11/1 |
Mathlib/RingTheory/DedekindDomain/Ideal.lean |
1 |
5 |
['Louddy', 'Ruben-VandeVelde', 'github-actions'] |
Ruben-VandeVelde assignee:Ruben-VandeVelde |
52-58334 1 month ago |
77-59604 2 months ago |
77-59657 77 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 |
27 |
['YaelDillies', 'b-mehta', 'eric-wieser', 'github-actions', 'kbuzzard', 'kmill', 'leanprover-community-mathlib4-bot'] |
kmill assignee:kmill |
52-58247 1 month ago |
99-32921 3 months ago |
147-52608 147 days |
24351 |
eric-wieser author:eric-wieser |
feat: fderiv lemmas for `pow` |
This generalizes the lemmas about `fderiv fun x => f x ^ n` to work over arbitrary normed modules and algebras.
Following the convention set by the lemmas about `fderiv` and `*`, we use `'`d names for the non-commutative variants.
Moves:
- `deriv_pow''` -> `deriv_pow`
- `deriv_pow` -> `deriv_pow_field`
- `derivWithin_pow'` -> `derivWithin_pow_field'`
Deletions:
- `deriv_pow'`
---
[](https://gitpod.io/from-referrer/)
|
t-analysis |
282/82 |
Mathlib.lean,Mathlib/Analysis/Calculus/Deriv/Polynomial.lean,Mathlib/Analysis/Calculus/Deriv/Pow.lean,Mathlib/Analysis/Calculus/FDeriv/Mul.lean,Mathlib/Analysis/Calculus/FDeriv/Pow.lean,Mathlib/Analysis/Calculus/Taylor.lean,Mathlib/Analysis/Complex/Angle.lean,Mathlib/Analysis/Convex/SpecificFunctions/Deriv.lean,Mathlib/NumberTheory/ModularForms/JacobiTheta/TwoVariable.lean |
9 |
2 |
['github-actions', 'leanprover-community-bot-assistant'] |
nobody |
51-12236 1 month ago |
51-12236 1 month ago |
51-45682 51 days |
24602 |
xyzw12345 author:xyzw12345 |
feat(LinearAlgebra/SymmetricAlgebra): IsSymmetricAlgebra |
This PR is a part of #21539, which separates out the part about `IsSymmetricAlgebra`.
Co-authored-by: Raphael Douglas Giles @Raph-DG
Co-authored-by: Zhixuan Dai <22300180006@m.fudan.edu.cn>
Co-authored-by: Zhenyan Fu
Co-authored-by: Yiming Fu
- [ ] depends on: #21539
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
78/0 |
Mathlib/LinearAlgebra/SymmetricAlgebra/Basic.lean,Mathlib/LinearAlgebra/SymmetricAlgebra/Basis.lean |
2 |
5 |
['eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
50-42100 1 month ago |
50-42352 1 month ago |
50-44292 50 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 |
50-31508 1 month ago |
50-37459 1 month ago |
98-3279 98 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 |
50-1501 1 month ago |
50-1501 1 month ago |
73-25620 73 days |
23497 |
chrisflav author:chrisflav |
chore(RingTheory/AdicCompletion/AsTensorProduct): golf using five lemma for modules |
---
- [x] depends on: #23496
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
30/81 |
Mathlib/RingTheory/AdicCompletion/AsTensorProduct.lean |
1 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
49-19239 1 month ago |
69-63596 2 months ago |
69-64420 69 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 |
48-78016 1 month ago |
49-256 1 month ago |
49-309 49 days |
24752 |
MichaelStollBayreuth author:MichaelStollBayreuth |
perf(Data.Real.Sqrt): make Real.sqrt irreducible |
We try to see what happens if we make `Real.sqrt` irreducible.
There are cases where this makes unification *very* significantly faster, compare [#mathlib4 > Coercion triggers timeout @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Coercion.20triggers.20timeout/near/517177117).
---
[](https://gitpod.io/from-referrer/)
|
t-data |
1/0 |
Mathlib/Data/Real/Sqrt.lean |
1 |
18 |
['MichaelStollBayreuth', 'eric-wieser', 'github-actions', 'leanprover-bot'] |
nobody |
48-33943 1 month ago |
50-47265 1 month ago |
50-52741 50 days |
24870 |
smmercuri author:smmercuri |
feat: `Field`, `FiniteDimensional` and `Algebra.IsSeparable` instances for `WithAbs` |
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-analysis
|
14/1 |
Mathlib/Analysis/Normed/Field/WithAbs.lean |
1 |
1 |
['github-actions'] |
nobody |
47-79398 1 month ago |
47-79405 1 month ago |
47-79548 47 days |
24872 |
smmercuri author:smmercuri |
feat: `apply` and `coe` results for `UniformSpace.Completion.mapRingHom` |
---
[](https://gitpod.io/from-referrer/)
|
t-topology |
9/0 |
Mathlib/Topology/Algebra/UniformRing.lean |
1 |
1 |
['github-actions'] |
nobody |
47-79177 1 month ago |
47-79177 1 month ago |
47-79224 47 days |
24883 |
madvorak author:madvorak |
chore(Data/Matrix): `Matrix.submatrix` naming convention |
I'm suggesting this change for the following reasons:
(1) managing expectations — `r_reindex` looks more like a propositional argument at first glance
(2) the original naming does not do justice to its motivation — there is nothing called `r` and `c` here — it would need to be `row_reindex` and `col_reindex` or something like that (if we wanted to use the convention for naming constants even tho we are naming a variable here)
---
Old version:
https://github.com/leanprover-community/mathlib4/pull/24135 |
t-data |
11/11 |
Mathlib/Data/Matrix/ConjTranspose.lean,Mathlib/Data/Matrix/Defs.lean |
2 |
1 |
['github-actions'] |
nobody |
47-75472 1 month ago |
47-75472 1 month ago |
47-75461 47 days |
24889 |
Kha author:Kha |
chore: do not include cache requests in build benchmark |
|
|
5/2 |
scripts/bench/temci-config.run.yml |
1 |
4 |
['Kha', 'github-actions', 'leanprover-bot'] |
nobody |
47-59391 1 month ago |
47-69226 1 month ago |
47-69208 47 days |
22153 |
smmercuri author:smmercuri |
feat: weak approximation theorems for infinite places of a number field |
The number field $K$ is dense in $\prod_v (K, v)$ and in the infinite adele ring $\prod_v K_v$, where $v$ ranges over the infinite places, $(K, v)$ denotes $K$ equipped with the topology induced by $v$, and $K_v$ is the completion of $K$ at $v$.
---
- [ ] depends on #22147
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-analysis
t-number-theory
label:t-algebra$ |
543/2 |
Mathlib/Algebra/Order/AbsoluteValue/Basic.lean,Mathlib/Analysis/AbsoluteValue/Equivalence.lean,Mathlib/Analysis/Normed/Ring/WithAbs.lean,Mathlib/NumberTheory/NumberField/AdeleRing.lean,Mathlib/NumberTheory/NumberField/InfinitePlace/Basic.lean |
5 |
1 |
['github-actions'] |
nobody |
47-56019 1 month ago |
47-73322 1 month ago |
59-10503 59 days |
24311 |
YaelDillies author:YaelDillies |
chore: replace `Monoid.IsTorsionFree` with `IsMulTorsionFree` |
From Toric
---
- [x] depends on: #24312
[](https://gitpod.io/from-referrer/)
|
toric
t-algebra
label:t-algebra$ |
63/29 |
Mathlib/Algebra/Group/Torsion.lean,Mathlib/Combinatorics/Additive/CauchyDavenport.lean,Mathlib/GroupTheory/Order/Min.lean,Mathlib/GroupTheory/Torsion.lean,Mathlib/Topology/Instances/ZMultiples.lean |
5 |
5 |
['YaelDillies', 'b-mehta', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
47-54546 1 month ago |
47-54546 1 month ago |
47-67875 47 days |
22043 |
YaelDillies author:YaelDillies |
chore: shortcut instance for `Neg ℤˣ` |
This lets us avoid importing `Ring` in downstream files (most of the effect is to come).
---
[](https://gitpod.io/from-referrer/)
|
file-removed
t-algebra
label:t-algebra$ |
20/47 |
Mathlib.lean,Mathlib/Algebra/GCDMonoid/Nat.lean,Mathlib/Algebra/Group/Int/Units.lean,Mathlib/Algebra/Order/Ring/Abs.lean,Mathlib/Algebra/Ring/Int/Units.lean,Mathlib/Algebra/Ring/NegOnePow.lean,Mathlib/Data/Fintype/Units.lean,Mathlib/Data/Int/AbsoluteValue.lean,Mathlib/Data/Int/Associated.lean,Mathlib/GroupTheory/HNNExtension.lean,Mathlib/NumberTheory/NumberField/Basic.lean,MathlibTest/Zify.lean |
12 |
15 |
['YaelDillies', 'eric-wieser', 'github-actions', 'j-loreaux', 'leanprover-community-bot-assistant', 'mathlib-bors'] |
nobody |
47-54289 1 month ago |
47-54289 1 month ago |
132-27324 132 days |
18379 |
oeb25 author:oeb25 |
feat(Topology/ENNReal): Add `ENNReal.tsum_biUnion` |
This adds infinite versions of `Finset.sum_biUnion` to `ENNReal`s.
---
One notable difference from the `Finset` version is that for `tsum` we have two ways for selecting the summands: `∑' x : ⋃ i ∈ S` or `∑' x : ⋃ i, t i`. This PR adds both.
I tried to extend this beyond `ENNReal`, but didn't find a clean way to do it.
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-topology
|
34/0 |
Mathlib/Data/Set/Lattice.lean,Mathlib/Data/Set/Pairwise/Lattice.lean,Mathlib/Topology/Instances/ENNReal/Lemmas.lean |
3 |
12 |
['github-actions', 'grunweg', 'j-loreaux', 'oeb25'] |
nobody |
46-63507 1 month ago |
46-64520 1 month ago |
149-26624 149 days |
24891 |
YaelDillies author:YaelDillies |
feat: `M ≃ₗ[R] (Fin (Module.finrank R M) → R)` for `M` a finite `R`-module |
From Toric
---
[](https://gitpod.io/from-referrer/)
|
toric
t-algebra
label:t-algebra$ |
13/3 |
Mathlib/LinearAlgebra/Dimension/Free.lean,Mathlib/LinearAlgebra/FreeModule/Basic.lean,Mathlib/LinearAlgebra/FreeModule/Finite/Basic.lean |
3 |
9 |
['YaelDillies', 'erdOne', 'eric-wieser', 'github-actions'] |
nobody |
46-41393 1 month ago |
47-51224 1 month ago |
47-68145 47 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 |
65/48 |
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/WithBot.lean,Mathlib/Probability/Moments/Variance.lean,Mathlib/RingTheory/PowerBasis.lean,Mathlib/Topology/MetricSpace/Holder.lean,Mathlib/Topology/MetricSpace/HolderNorm.lean |
14 |
20 |
['YaelDillies', 'b-mehta', 'eric-wieser', 'github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'urkud'] |
nobody |
44-74416 1 month ago |
44-74437 1 month ago |
94-66989 94 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 |
43-68969 1 month ago |
59-68609 1 month ago |
59-76523 59 days |
19796 |
peakpoint author:peakpoint |
feat: L'Hopital's rule from within a convex set |
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-analysis
|
190/19 |
Mathlib/Algebra/Polynomial/Module/Basic.lean,Mathlib/Analysis/Calculus/LHopital.lean,Mathlib/Analysis/Convex/Topology.lean,Mathlib/Geometry/Manifold/Instances/Real.lean,Mathlib/Order/Interval/Set/Basic.lean |
5 |
14 |
['RemyDegenne', 'github-actions', 'leanprover-community-bot-assistant', 'peakpoint', 'sgouezel'] |
sgouezel assignee:sgouezel |
43-22848 1 month ago |
43-22848 1 month ago |
76-59531 76 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 |
11 |
['eric-wieser', 'github-actions', 'madvorak'] |
nobody |
42-50266 1 month ago |
50-55111 1 month ago |
52-4939 52 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 |
42-39765 1 month ago |
42-39889 1 month ago |
42-43353 42 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$ |
215/155 |
Mathlib/Algebra/Algebra/Operations.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Affine/Point.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 |
8 |
7 |
['alreadydone', 'github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
41-69076 1 month ago |
41-69231 1 month ago |
118-38359 118 days |
22631 |
Thmoas-Guan author:Thmoas-Guan |
feat(Algebra): define associated graded structure for abelian group |
In this PR we define the associated graded structure for abelian group when given a filtration and only give some basic lemmas about it.
Further results would be given in #20913
---
- [x] depends on: #24071
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
155/0 |
Mathlib.lean,Mathlib/RingTheory/FilteredAlgebra/AssociatedGraded.lean |
2 |
17 |
['AntoineChambert-Loir', 'Thmoas-Guan', 'eric-wieser', 'github-actions', 'kbuzzard', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
41-65422 1 month ago |
41-65442 1 month ago |
116-23622 116 days |
25044 |
alreadydone author:alreadydone |
feat(Topology/Algebra): `Homeomorph` version of `unitsEquivNeZero` |
also add `Topology.IsEmbedding.homeomorphImage`: a set is homeomorphic to its image under any embedding.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-topology
label:t-algebra$ |
51/28 |
Mathlib/Topology/Algebra/GroupWithZero.lean,Mathlib/Topology/Homeomorph/Lemmas.lean |
2 |
1 |
['github-actions'] |
nobody |
41-58168 1 month ago |
41-62423 1 month ago |
41-62406 41 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 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
41-40597 1 month ago |
41-48352 1 month ago |
41-49731 41 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 |
40-11986 1 month ago |
68-9543 2 months ago |
68-9596 68 days |
16074 |
Rida-Hamadani author:Rida-Hamadani |
feat: combinatorial maps and planar graphs |
We define combinatorial maps, then we define planar graph using combinatorial maps.
---
[](https://gitpod.io/from-referrer/)
|
t-combinatorics |
243/0 |
Mathlib.lean,Mathlib/Combinatorics/SimpleGraph/Planar.lean,Mathlib/Data/CombinatorialMap.lean |
3 |
27 |
['Parcly-Taxel', 'Rida-Hamadani', 'github-actions', 'lambda-fairy', 'leanprover-community-bot-assistant'] |
kmill assignee:kmill |
39-54326 1 month ago |
64-65928 2 months ago |
68-53358 68 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 |
39-54177 1 month ago |
75-65563 2 months ago |
131-26284 131 days |
25101 |
erdOne author:erdOne |
feat(AlgebraicGeometry): building morphisms into Proj |
---
[](https://gitpod.io/from-referrer/)
|
t-algebraic-geometry |
231/3 |
Mathlib/AlgebraicGeometry/ProjectiveSpectrum/Basic.lean,Mathlib/AlgebraicGeometry/Restrict.lean,Mathlib/AlgebraicGeometry/Scheme.lean,Mathlib/RingTheory/GradedAlgebra/HomogeneousLocalization.lean |
4 |
6 |
['erdOne', 'github-actions', 'joelriou'] |
nobody |
39-22285 1 month ago |
39-22285 1 month ago |
40-1973 40 days |
25123 |
eric-wieser author:eric-wieser |
feat: add rfl lemmas for monoidal categories |
Making these `simp` opens a can of worms best left to #24823
`simps` would generate bad names here.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
111/0 |
Mathlib/Algebra/Category/AlgCat/Monoidal.lean,Mathlib/Algebra/Category/ModuleCat/Monoidal/Basic.lean,Mathlib/LinearAlgebra/QuadraticForm/QuadraticModuleCat/Monoidal.lean |
3 |
1 |
['github-actions'] |
nobody |
39-11793 1 month ago |
39-11793 1 month ago |
39-11845 39 days |
23365 |
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/)
|
large-import
t-meta
|
440/73 |
Mathlib/Tactic/Simproc/ExistsAndEq.lean,MathlibTest/Simproc/ExistsAndEq.lean |
2 |
41 |
['JovanGerb', 'b-mehta', 'eric-wieser', 'github-actions', 'grunweg', 'kim-em', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'vasnesterov'] |
nobody |
38-66669 1 month ago |
89-17754 2 months ago |
94-44394 94 days |
24528 |
chrisflav author:chrisflav |
feat(AlgebraicGeometry): directed covers |
Directed covers are covers, where every intersection can be covered by a component of the cover. For open covers this is equivalent to the images forming a basis of the topology.
If a cover is directed, the compatibility conditions for gluing become easier, because only compatibility with the transition maps needs to be checked.
---
[](https://gitpod.io/from-referrer/)
|
t-algebraic-geometry |
233/0 |
Mathlib.lean,Mathlib/AlgebraicGeometry/Cover/Directed.lean |
2 |
6 |
['chrisflav', 'erdOne', 'github-actions', 'joelriou', 'leanprover-community-bot-assistant'] |
nobody |
38-55659 1 month ago |
38-55726 1 month ago |
55-40749 55 days |
25069 |
erdOne author:erdOne |
feat(EllipticCurve): rational points of singular nodal cubics |
---
[](https://gitpod.io/from-referrer/)
|
t-algebraic-geometry |
251/0 |
Mathlib.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Affine/Basic.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Singular/Node.lean |
3 |
11 |
['Multramate', 'acmepjz', 'erdOne', 'github-actions'] |
nobody |
38-46999 1 month ago |
41-7501 1 month ago |
41-7557 41 days |
25071 |
erdOne author:erdOne |
feat(EllipticCurve): basic API for singular cubics |
---
[](https://gitpod.io/from-referrer/)
|
t-algebraic-geometry |
320/0 |
Mathlib.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Singular/Basic.lean,Mathlib/AlgebraicGeometry/EllipticCurve/VariableChange.lean |
3 |
34 |
['Multramate', 'acmepjz', 'erdOne', 'github-actions'] |
nobody |
38-3835 1 month ago |
41-5658 1 month ago |
41-5713 41 days |
24103 |
plp127 author:plp127 |
feat(Topology/UniformSpace/OfCompactT2): generalize theorem |
Generalize `uniformSpaceOfCompactT2` to `uniformSpaceOfCompactR1`.
---
- [ ] depends on: #24098
[](https://gitpod.io/from-referrer/)
|
t-topology |
48/24 |
Mathlib/Topology/Separation/Regular.lean,Mathlib/Topology/UniformSpace/OfCompactT2.lean |
2 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
36-33254 1 month ago |
36-33276 1 month ago |
68-23234 68 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 |
35-40678 1 month ago |
77-28976 2 months ago |
77-29027 77 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 |
35-31133 1 month ago |
41-7534 1 month ago |
41-7530 41 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 |
3 |
['github-actions', 'leanprover-community-bot-assistant'] |
ericrbg assignee:ericrbg |
34-56804 1 month ago |
34-56821 1 month ago |
112-78569 112 days |
23684 |
alreadydone author:alreadydone |
feat(RingTheory): integral extensions of comm. rings are local homs |
---
The import increase only affects one file so I hope it's okay.
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebra
label:t-algebra$ |
57/65 |
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/RingTheory/Artinian/Ring.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 |
13 |
4 |
['alreadydone', 'github-actions', 'xroblot'] |
nobody |
34-36919 1 month ago |
87-15911 2 months ago |
87-15930 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'] |
nobody |
34-26816 1 month ago |
35-18228 1 month ago |
35-18284 35 days |
25248 |
xcloudyunx author:xcloudyunx |
feat(Combinatorics/SimpleGraph): Add Subgraph.inclusion_edge_apply_coe and inclusion_edgeSet_apply_coe |
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-combinatorics
|
12/0 |
Mathlib/Combinatorics/SimpleGraph/Subgraph.lean |
1 |
1 |
['github-actions'] |
nobody |
34-20458 1 month ago |
34-20459 1 month ago |
34-20513 34 days |
25238 |
Hagb author:Hagb |
feat(Tactic/ComputeDegree): add support for scalar multiplication with different types |
It would be able to deal with `a • (X : R[X])` where `a : S` is in a different type `S` with `[SMulZeroClass S R]`.
---
- [x] depends on: #25237
[](https://gitpod.io/from-referrer/)
|
new-contributor |
17/5 |
Mathlib/Tactic/ComputeDegree.lean,MathlibTest/ComputeDegree.lean |
2 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
34-448 1 month ago |
34-24891 1 month ago |
34-26793 34 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 |
33-78406 1 month ago |
37-44145 1 month ago |
37-44127 37 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 |
33-73084 1 month ago |
34-49026 1 month ago |
40-53421 40 days |
25179 |
YaelDillies author:YaelDillies |
feat: `#track_sorry`, a command to find usage of `sorry` |
`#track_sorry foo` returns a non-sorry-free declaration `bar` which `foo` depends on, if such `bar` exists.
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
---
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
|
71/0 |
Mathlib.lean,Mathlib/Util/TrackSorry.lean |
2 |
11 |
['YaelDillies', 'eric-wieser', 'github-actions', 'kmill'] |
nobody |
33-63193 1 month ago |
36-72008 1 month ago |
36-72061 36 days |
25271 |
YaelDillies author:YaelDillies |
feat: promote an `AlgEquiv` preserving `counit` and `comul` to a `BialgEquiv` |
From Toric
---
[](https://gitpod.io/from-referrer/)
|
toric
t-algebra
label:t-algebra$ |
38/24 |
Mathlib/Algebra/Algebra/Equiv.lean,Mathlib/Algebra/Algebra/Hom.lean,Mathlib/RingTheory/Bialgebra/Equiv.lean |
3 |
1 |
['github-actions'] |
nobody |
33-36523 1 month ago |
33-40172 1 month ago |
33-40166 33 days |
24412 |
pechersky author:pechersky |
feat(UniformSpace/Ultra/Constructions): IsUltraUniformity.{bot,top} |
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-topology
|
29/0 |
Mathlib/Order/Filter/Bases/Basic.lean,Mathlib/Topology/UniformSpace/Defs.lean,Mathlib/Topology/UniformSpace/Ultra/Basic.lean,Mathlib/Topology/UniformSpace/Ultra/Constructions.lean |
4 |
6 |
['github-actions', 'pechersky', 'urkud'] |
urkud assignee:urkud |
33-7797 1 month ago |
33-11007 1 month ago |
58-7966 58 days |
25273 |
YaelDillies author:YaelDillies |
feat: `Finsupp.linearCombination MonoidAlgebra.of = id` |
From Toric
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebra
label:t-algebra$ |
8/1 |
Mathlib/Algebra/MonoidAlgebra/Defs.lean |
1 |
4 |
['YaelDillies', 'eric-wieser', 'github-actions'] |
nobody |
32-70205 1 month ago |
33-38345 1 month ago |
33-38393 33 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 |
32-37195 1 month ago |
32-37195 1 month ago |
32-55579 32 days |
21950 |
erdOne author:erdOne |
feat(NumberTheory/Padics): the completion of `ℚ` at a finite place is `ℚ_[p]` |
---
[](https://gitpod.io/from-referrer/)
|
t-number-theory |
253/1 |
Mathlib.lean,Mathlib/Algebra/GroupWithZero/WithZero.lean,Mathlib/NumberTheory/Padics/HeightOneSpectrum.lean,Mathlib/NumberTheory/Padics/PadicNumbers.lean,Mathlib/Topology/Algebra/Valued/WithVal.lean,Mathlib/Topology/Algebra/WithZeroMulInt.lean,Mathlib/Topology/Algebra/WithZeroTopology.lean |
7 |
22 |
['Ruben-VandeVelde', 'erdOne', 'github-actions', 'leanprover-community-bot-assistant', 'pechersky', 'smmercuri', 'xroblot'] |
nobody |
31-12608 1 month ago |
31-12608 1 month ago |
72-51603 72 days |
25322 |
thorimur author:thorimur |
style: use simplex notation (`⦋n⦌`) where possible |
`StandardSimplex.mk n` is replaced with `⦋n⦌` where possible (except in notation and macros, which are left untouched). This includes opening `Simplicial` in two files. Also, outdated and unused `local notation` `[n]` for `StandardSimplex.mk n` is removed.
---
[](https://gitpod.io/from-referrer/)
|
t-topology |
38/39 |
Mathlib/AlgebraicTopology/CechNerve.lean,Mathlib/AlgebraicTopology/MooreComplex.lean,Mathlib/AlgebraicTopology/SimplexCategory/Basic.lean,Mathlib/AlgebraicTopology/SimplicialObject/Basic.lean,Mathlib/AlgebraicTopology/SimplicialSet/Coskeletal.lean,Mathlib/AlgebraicTopology/SimplicialSet/NerveAdjunction.lean,Mathlib/AlgebraicTopology/SimplicialSet/StdSimplex.lean |
7 |
1 |
['github-actions'] |
nobody |
31-9645 1 month ago |
31-20224 1 month ago |
31-20276 31 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 |
9 |
['YaelDillies', 'erdOne', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant'] |
nobody |
30-41588 1 month ago |
30-41607 1 month ago |
33-40338 33 days |
25284 |
alreadydone author:alreadydone |
feat(LinearAlgebra/Contraction): bijectivity of `dualTensorHom` + generalize to CommSemiring |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
168/44 |
Mathlib/Data/Finsupp/Defs.lean,Mathlib/LinearAlgebra/Contraction.lean,Mathlib/LinearAlgebra/Pi.lean,Mathlib/LinearAlgebra/Trace.lean,Mathlib/RingTheory/Finiteness/Finsupp.lean |
5 |
5 |
['alreadydone', 'eric-wieser', 'github-actions', 'leanprover-bot'] |
nobody |
30-21034 1 month ago |
33-23406 1 month ago |
33-23390 33 days |
25343 |
plp127 author:plp127 |
docs(Topology/Perfect): Mention dense-in-itself |
The file `Mathlib/Topology/Perfect` defines a "nonstandard" predicate `Preperfect C` to mean that every point of `C` is an accumulation point of `C`. This property already has a name, it is called [dense-in-itself](https://en.wikipedia.org/wiki/Dense-in-itself). This PR adds this name to the docs.
---
[](https://gitpod.io/from-referrer/)
|
t-topology
documentation
|
7/7 |
Mathlib/Topology/Perfect.lean |
1 |
1 |
['github-actions'] |
nobody |
29-57421 29 days ago |
29-57499 29 days ago |
29-57483 29 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 |
29-5858 29 days ago |
30-15580 1 month ago |
30-15570 30 days |
22069 |
Raph-DG author:Raph-DG |
feat(LinearMap): Added lemmas relating kernels of linear maps to Submodule.map |
Added the lemma ne_map_or_ne_kernel_inter_of_lt stating that if A < B as submodules, then for any linear map f, `ker f ⊓ A ≠ ker f ⊓ B ∨ Submodule.map f A ≠ Submodule.map f B`. We also prove the corollaries ker_inter_mono_of_map_eq and map_mono_of_ker_inter_eq.
Co-authored-by: Raphael Douglas Giles (raphaeldouglasgiles@gmail.com)
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-algebra
label:t-algebra$ |
30/0 |
Mathlib/LinearAlgebra/Span/Basic.lean |
1 |
21 |
['Paul-Lez', 'Raph-DG', 'github-actions', 'j-loreaux', 'mattrobball'] |
mattrobball assignee:mattrobball |
28-61192 28 days ago |
28-61192 28 days ago |
131-14482 131 days |
24884 |
smmercuri author:smmercuri |
feat: `ramificationIdx` for `NumberField.InfinitePlace` |
---
- [x] depends on: #24880
[](https://gitpod.io/from-referrer/)
|
t-number-theory |
38/0 |
Mathlib/NumberTheory/NumberField/InfinitePlace/Ramification.lean |
1 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'riccardobrasca'] |
nobody |
27-49512 27 days ago |
42-54230 1 month ago |
42-54577 42 days |
24875 |
smmercuri author:smmercuri |
feat: injectivity of `InfinitePlace.embedding` |
---
[](https://gitpod.io/from-referrer/)
|
t-number-theory |
19/0 |
Mathlib/NumberTheory/NumberField/InfinitePlace/Basic.lean |
1 |
6 |
['Ruben-VandeVelde', 'github-actions', 'riccardobrasca', 'smmercuri', 'xroblot'] |
nobody |
26-65112 26 days ago |
47-78702 1 month ago |
47-78755 47 days |
25410 |
JovanGerb author:JovanGerb |
chore: remove some duplicate instances |
I have a program that finds duplicate instances, as described at [#mathlib4 > duplicate declarations](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/duplicate.20declarations/with/518941841)
This PR is a start at fixing these in Mathlib.
---
[](https://gitpod.io/from-referrer/)
|
|
30/131 |
Mathlib/Algebra/Category/Grp/Adjunctions.lean,Mathlib/Algebra/Category/ModuleCat/Basic.lean,Mathlib/Algebra/Group/Fin/Basic.lean,Mathlib/Algebra/Homology/Embedding/IsSupported.lean,Mathlib/Algebra/Order/Hom/Monoid.lean,Mathlib/Algebra/Ring/Divisibility/Basic.lean,Mathlib/Algebra/Ring/Subsemiring/Basic.lean,Mathlib/AlgebraicGeometry/Limits.lean,Mathlib/AlgebraicGeometry/OpenImmersion.lean,Mathlib/CategoryTheory/Countable.lean,Mathlib/CategoryTheory/EffectiveEpi/Preserves.lean,Mathlib/CategoryTheory/ObjectProperty/FullSubcategory.lean,Mathlib/Computability/TuringDegree.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/Data/Fintype/EquivFin.lean,Mathlib/Data/List/TakeDrop.lean,Mathlib/Data/Matroid/Constructions.lean,Mathlib/Data/Nat/Basic.lean,Mathlib/Data/Option/Defs.lean,Mathlib/Data/Ordering/Basic.lean,Mathlib/Data/Sign.lean,Mathlib/GroupTheory/Perm/Sign.lean,Mathlib/GroupTheory/Solvable.lean,Mathlib/Logic/Embedding/Basic.lean,Mathlib/Logic/Equiv/Fin/Basic.lean,Mathlib/ModelTheory/Basic.lean,Mathlib/Order/Monotone/Basic.lean,Mathlib/SetTheory/Cardinal/Basic.lean,Mathlib/Tactic/Polyrith.lean,Mathlib/Topology/Compactness/Lindelof.lean |
30 |
9 |
['JovanGerb', 'adomani', 'eric-wieser', 'github-actions'] |
nobody |
26-61536 26 days ago |
27-20789 27 days ago |
27-20772 27 days |
25401 |
digama0 author:digama0 |
feat(Util): SuppressSorry option |
See also leanprover/lean4#8611 and [#lean4 > Silent sorry @ 💬](https://leanprover.zulipchat.com/#narrow/channel/270676-lean4/topic/Silent.20sorry/near/503537964). This is a stop-gap solution while leanprover/lean4#8611 is underway, but it works about as well as any other built in option. Hooking declaration elaborators turns out to be a very powerful technique.
---
[](https://gitpod.io/from-referrer/)
|
t-meta |
342/0 |
Mathlib.lean,Mathlib/Util/CommandElabHook.lean,Mathlib/Util/SuppressSorry.lean,MathlibTest/suppressSorry.lean |
4 |
13 |
['digama0', 'eric-wieser', 'github-actions'] |
nobody |
26-11851 26 days ago |
26-36185 26 days ago |
27-46534 27 days |
25453 |
JovanGerb author:JovanGerb |
perf(Algebra/Homology/HomotopyCategory): use explicit universe parameter in `Category` |
As we have seen before, writing `Category.{v}` instead of `Category` avoids a nasty universe level metavariable, and this helps to speed up unification. The changes in this PR are somewhat arbitrary, but it serves as an example for this principle.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
9/6 |
Mathlib/Algebra/Homology/HomotopyCategory/DegreewiseSplit.lean,Mathlib/Algebra/Homology/HomotopyCategory/MappingCone.lean,Mathlib/Algebra/Homology/HomotopyCategory/Triangulated.lean |
3 |
5 |
['JovanGerb', 'github-actions', 'leanprover-bot'] |
nobody |
25-62839 25 days ago |
26-30487 26 days ago |
26-30540 26 days |
25265 |
FMLJohn author:FMLJohn |
feat(Order/SupClosed): `compl_image_latticeClosure` and `compl_image_latticeClosure_eq_of_compl_image_eq_self` |
The main results in this pull request are:
1. `compl_image_latticeClosure`: given any Boolean algebra `α` and `s : Set α`, `compl '' latticeClosure s` is the same as `latticeClosure (compl '' s)`;
2. `compl_image_latticeClosure_eq_of_compl_image_eq_self`: given any Boolean algebra `α` and `s : Set α` such that `compl '' s = s`, we have `compl '' latticeClosure s = latticeClosure s`.
---
[](https://gitpod.io/from-referrer/) |
maintainer-merge
t-order
|
59/1 |
Mathlib/Order/SupClosed.lean |
1 |
8 |
['FMLJohn', 'YaelDillies', 'github-actions'] |
bryangingechen assignee:bryangingechen |
25-52263 25 days ago |
28-32235 28 days ago |
32-41854 32 days |
25483 |
VTrelat author:VTrelat |
chore(Data/Set/Prod, SetTheory/ZFC/Basic): add theorem prod_subset_of_prod and extend ZFC model |
Required by @eric-wieser in #24281
---
[](https://gitpod.io/from-referrer/)
|
t-data
new-contributor
|
103/0 |
Mathlib/Data/Set/Prod.lean,Mathlib/SetTheory/ZFC/Basic.lean |
2 |
2 |
['VTrelat', 'github-actions'] |
nobody |
25-50275 25 days ago |
25-56894 25 days ago |
25-56947 25 days |
25450 |
pechersky author:pechersky |
feat(Valued): Valuation.leAddSubgroup and ideal/submodule versions of ltAddSubgroup |
Also prove that these are clopen.
Factored out of #24627
Fix capitalization spelling mistake on `closedball` in a lemma
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-analysis
t-number-theory
label:t-algebra$ |
272/30 |
Mathlib/RingTheory/Valuation/Basic.lean,Mathlib/RingTheory/Valuation/Integers.lean,Mathlib/Topology/Algebra/Valued/LocallyCompact.lean,Mathlib/Topology/Algebra/Valued/ValuationTopology.lean |
4 |
4 |
['faenuccio', 'github-actions', 'pechersky'] |
nobody |
25-37 25 days ago |
26-35961 26 days ago |
26-37479 26 days |
25089 |
Bergschaf author:Bergschaf |
feat(Order/Sublocale): definition of sublocales |
There are several possible definition of sublocales. I used one from [nlab](https://ncatlab.org/nlab/show/sublocale) which states that a sublocale is a subset of a locale which is closed under all meets and for any ∈ S and x ∈ X, we have x ⇨ s ∈ S.
This PR also includes an order isomorphism between (Nucleus)ᵒᵈ and Sublocale.
---
I am open to better name suggestions for the order isomorphism.
- [x] depends on: #24941
[](https://gitpod.io/from-referrer/)
|
maintainer-merge
t-order
|
265/8 |
Mathlib.lean,Mathlib/Order/Hom/Lattice.lean,Mathlib/Order/Nucleus.lean,Mathlib/Order/Sublocale.lean,Mathlib/Order/Synonym.lean,docs/references.bib |
6 |
71 |
['Bergschaf', 'YaelDillies', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'xhalo32'] |
nobody |
23-31069 23 days ago |
23-31069 23 days ago |
37-10491 37 days |
25481 |
kbuzzard author:kbuzzard |
chore: refactor Algebra.TensorProduct.rightAlgebra |
The declaration `Algebra.TensorProduct.rightAlgebra` makes `A ⊗[R] B` into a `B`-algebra (here `R` is a `CommSemiring`, `A` is a `Semiring` and an `R`-algebra, and `B` is a `CommSemiring` and an `R`-algebra). It is not an instance because if A = B it causes a diamond. However in the many cases where A isn't B, it can occasionally be useful.
However one could imagine that in the many cases where an R-module `M` also isn't `B`, it might occasionally be useful to make `M ⊗[R] B` into a `B`-module (and indeed I am finding this in FLT). With the current definition of `Algebra.TensorProduct.rightAlgebra` this is difficult to do without causing diamonds in the case when `M` happens to be an `R`-algebra (by which I mean "I failed to do this in finite time").
One fix for this is just to redefine `Algebra.TensorProduct.rightAlgebra` so that the `smul` field is
```
smul b ab := TensorProduct.comm _ _ _ (b • (TensorProduct.comm _ _ _ ab))
```
i.e. literally "swap the product around, use mathlib's instance making `B ⊗[R] A` into a `B`-algebra, and then swap back". Then the same definition can be used to make `M ⊗[R] B` into a `B`-module and on the odd occasion where this point of view is useful, there is no diamond. This is what we do in this PR. After adding one simp lemma there is no breakage at all in mathlib. Furthermore, for those who have observed that we want to build on this algebra instance sometimes and, for example, add instances of the form "if M is finite over R then M ⊗[R] B is finite over B" -- these instances are really easy to add now with this new definition, because you simply pull back the analogous finite left module instance along the isomorphism M ⊗[R] B = B ⊗[R] M. Examples (from FLT, where the right action is put in a scope):
```
scoped instance [Module.Finite R M] : Module.Finite A (M ⊗[R] A) :=
Module.Finite.equiv (Module.TensorProduct.comm R A M)
scoped instance [Module.Free R M] : Module.Free A (M ⊗[R] A) :=
Module.Free.of_equiv (Module.TensorProduct.comm R A M)
```
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
33/6 |
Mathlib/RingTheory/TensorProduct/Basic.lean |
1 |
4 |
['github-actions', 'kbuzzard', 'leanprover-bot'] |
nobody |
22-73856 22 days ago |
25-53403 25 days ago |
25-53660 25 days |
25563 |
Komyyy author:Komyyy |
chore: move `Topology.StoneCech` into `Topology.Compactification` (1/2) |
At present, the `Topology.Compactification` directory includes results on one-point compactifications, but results on Stone-Čech compactifications are currently located elsewhere.
The removed file `Topology.Compactification` is deprecated in another PR (#25583) to leave a good git diff history.
---
[](https://gitpod.io/from-referrer/)
|
file-removed
maintainer-merge
t-topology
|
9/9 |
Mathlib.lean,Mathlib/Combinatorics/Hindman.lean,Mathlib/Topology/Category/CompHaus/Basic.lean,Mathlib/Topology/Category/CompHaus/Projective.lean,Mathlib/Topology/Category/Profinite/Projective.lean,Mathlib/Topology/Category/Stonean/Adjunctions.lean,Mathlib/Topology/Compactification/StoneCech.lean,Mathlib/Topology/ExtremallyDisconnected.lean,Mathlib/Topology/Maps/Proper/UniversallyClosed.lean,Mathlib/Topology/Separation/CompletelyRegular.lean |
10 |
4 |
['Komyyy', 'github-actions', 'grunweg'] |
nobody |
22-72225 22 days ago |
22-72225 22 days ago |
23-47757 23 days |
25578 |
peakpoint author:peakpoint |
refactor(Geometry/Euclidean/Projection): redefine projection and reflection for affine subspaces |
---
The coersion stuff is just copied from `Analysis/Normed/Operator/LinearIsometry`.
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-euclidean-geometry
|
479/448 |
Mathlib.lean,Mathlib/Analysis/Normed/Affine/ContinuousAffineMap.lean,Mathlib/Analysis/Normed/Affine/Isometry.lean,Mathlib/Geometry/Euclidean/Altitude.lean,Mathlib/Geometry/Euclidean/Circumcenter.lean,Mathlib/Geometry/Euclidean/Projection.lean,Mathlib/Geometry/Euclidean/SignedDist.lean,Mathlib/LinearAlgebra/AffineSpace/AffineSubspace/Projection.lean |
8 |
2 |
['github-actions', 'jsm28'] |
nobody |
22-59387 22 days ago |
23-8287 23 days ago |
23-8282 23 days |
24541 |
pfaffelh author:pfaffelh |
feat(Topology/Compactness/CompactSystem): introduce compact Systems |
A compact system is a set systems with the property that, whenever a countable intersections of sets in the set system is empty, there is a finite subset of sets with empty intersection. These are needed e.g. in measure theory if one wants to show sigma-additivity of a set function on a ring.
* Main result: The set of sets which are either compact and closed, or `univ`, is a compact system.
* Introduce `Dissipate s x := ⋂ y ≤ x, s y` (Data/Set/Dissipate), which is parallel to Data/Set/Accumulate.
Co-authored-by: Rémy Degenne remydegenne@gmail.com
|
new-contributor
t-measure-probability
|
453/2 |
Mathlib.lean,Mathlib/Data/Set/Accumulate.lean,Mathlib/Data/Set/Dissipate.lean,Mathlib/MeasureTheory/PiSystem.lean,Mathlib/Topology/Compactness/CompactSystem.lean |
5 |
74 |
['github-actions', 'leanprover-community-bot-assistant', 'pfaffelh', 'sgouezel'] |
nobody |
22-37551 22 days ago |
22-37551 22 days ago |
41-71364 41 days |
25600 |
Komyyy author:Komyyy |
refactor: lemma expressing `ContinuousAt` using a punctured neighbourhood |
---
This lemma is used to prove that the Riemann zeta function is meromorphic in #25597.
[](https://gitpod.io/from-referrer/)
|
maintainer-merge
t-topology
|
4/0 |
Mathlib/Topology/ContinuousOn.lean |
1 |
5 |
['Komyyy', 'github-actions', 'grunweg'] |
nobody |
22-22942 22 days ago |
22-22942 22 days ago |
22-34829 22 days |
25573 |
JovanGerb author:JovanGerb |
feat: define `∃ x > y, ...` notation to mean `∃ x, y < x ∧ ...` |
This PR changes the elaboration of the binders `∃ x > y,` and `∀ x > y,` to use `<` instead of `>`, because we want to avoid working with `>` as much as possible (and similarly for `≥` vs `≤` ).
The advantage is that we don't need to worry about rewriting with lemmas like `gt_iff_lt`. The disadvantage is that people might find this confusing.
[#mathlib4 > naming convention for ≤ and < @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/naming.20convention.20for.20.E2.89.A4.20and.20.3C/near/522910464)
The main changes are in `Mathlib.Init`, `Mathlib.Util.Delaborators` and `MathlibTest.delaborators`.
---
[](https://gitpod.io/from-referrer/)
|
t-meta |
59/52 |
Counterexamples/DiscreteTopologyNonDiscreteUniformity.lean,Mathlib/Algebra/Order/Monoid/Canonical/Defs.lean,Mathlib/Analysis/Analytic/Basic.lean,Mathlib/Analysis/BoxIntegral/Integrability.lean,Mathlib/Analysis/Calculus/UniformLimitsDeriv.lean,Mathlib/Analysis/Complex/Liouville.lean,Mathlib/Analysis/Complex/OpenMapping.lean,Mathlib/Analysis/Fourier/PoissonSummation.lean,Mathlib/Analysis/MellinTransform.lean,Mathlib/Analysis/Normed/Operator/Banach.lean,Mathlib/Dynamics/Ergodic/Conservative.lean,Mathlib/Dynamics/PeriodicPts/Defs.lean,Mathlib/Geometry/Manifold/IntegralCurve/ExistUnique.lean,Mathlib/Init.lean,Mathlib/MeasureTheory/Covering/LiminfLimsup.lean,Mathlib/MeasureTheory/Function/ConvergenceInMeasure.lean,Mathlib/MeasureTheory/Function/Egorov.lean,Mathlib/MeasureTheory/Function/StronglyMeasurable/Basic.lean,Mathlib/MeasureTheory/Integral/DivergenceTheorem.lean,Mathlib/MeasureTheory/Integral/Layercake.lean,Mathlib/NumberTheory/LSeries/SumCoeff.lean,Mathlib/Order/Filter/AtTopBot/Finite.lean,Mathlib/RingTheory/RootsOfUnity/PrimitiveRoots.lean,Mathlib/RingTheory/Valuation/Basic.lean,Mathlib/Topology/CWComplex/Classical/Finite.lean,Mathlib/Topology/ContinuousMap/Ideals.lean,Mathlib/Topology/EMetricSpace/Defs.lean,Mathlib/Topology/EMetricSpace/Paracompact.lean,Mathlib/Topology/LocallyFinite.lean,Mathlib/Topology/MetricSpace/Ultra/Basic.lean,Mathlib/Util/Delaborators.lean,MathlibTest/delaborators.lean |
32 |
1 |
['github-actions'] |
nobody |
22-18238 22 days ago |
22-18350 22 days ago |
22-18338 22 days |
22603 |
pechersky author:pechersky |
chore(Topology): rename pi family from π to X |
Only in files that mentioned such a family, via a script:
```
git grep -e "π : . → Type" --name-only | rg Topology | xargs -I{} sed -i -e 's/π/X/g' {}
```
---
[](https://gitpod.io/from-referrer/)
|
tech debt
t-topology
|
238/238 |
Mathlib/Topology/AlexandrovDiscrete.lean,Mathlib/Topology/Algebra/InfiniteSum/Constructions.lean,Mathlib/Topology/Algebra/Module/Equiv.lean,Mathlib/Topology/Algebra/Order/LiminfLimsup.lean,Mathlib/Topology/Bases.lean,Mathlib/Topology/Bornology/Constructions.lean,Mathlib/Topology/Connected/Basic.lean,Mathlib/Topology/Connected/Clopen.lean,Mathlib/Topology/Connected/LocallyConnected.lean,Mathlib/Topology/Connected/TotallyDisconnected.lean,Mathlib/Topology/Constructions.lean,Mathlib/Topology/ContinuousOn.lean,Mathlib/Topology/EMetricSpace/Diam.lean,Mathlib/Topology/EMetricSpace/Pi.lean,Mathlib/Topology/ExtremallyDisconnected.lean,Mathlib/Topology/Inseparable.lean,Mathlib/Topology/MetricSpace/Basic.lean,Mathlib/Topology/MetricSpace/Infsep.lean,Mathlib/Topology/MetricSpace/ProperSpace.lean,Mathlib/Topology/MetricSpace/Pseudo/Pi.lean,Mathlib/Topology/Metrizable/Basic.lean,Mathlib/Topology/Order/Basic.lean,Mathlib/Topology/Separation/Hausdorff.lean,Mathlib/Topology/UniformSpace/Ascoli.lean |
24 |
1 |
['github-actions'] |
nobody |
22-9988 22 days ago |
22-10010 22 days ago |
28-3624 28 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$ |
92/1 |
Mathlib.lean,Mathlib/Algebra/Ring/Equiv.lean,Mathlib/RingTheory/RingHom/FaithfullyFlat.lean,Mathlib/RingTheory/RingHom/Flat.lean |
4 |
4 |
['chrisflav', 'erdOne', 'github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
21-72326 21 days ago |
51-66334 1 month ago |
51-67399 51 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 |
4 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
21-69618 21 days ago |
21-72314 21 days ago |
21-73254 21 days |
24520 |
chrisflav author:chrisflav |
feat(Algebra/Pi): add various `AlgEquiv`s and `RingEquiv`s |
Add
- `RingEquiv.sumArrowEquivProdArrow`: ring version of `Equiv.sumArrowEquivProdArrow`.
- `AlgEquiv.sumArrowEquivProdArrow`: algebra version of `Equiv.sumArrowEquivProdArrow`.
- `AlgEquiv.piCongrLeft'`: algebra version of `Equiv.piCongrLeft`.
- `AlgEquiv.piCongrLeft`: algebra version of `Equiv.piCongrLeft`.
- `AlgEquiv.funUnique`: algebra version of `Equiv.funUnique`.
- `AlgEquiv.prodCongr`: algebra version of `Equiv.prodCongr`.
The four last ones already have ring versions.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
116/1 |
Mathlib/Algebra/Algebra/Pi.lean,Mathlib/Algebra/Algebra/Prod.lean,Mathlib/Algebra/Ring/Equiv.lean |
3 |
20 |
['Ruben-VandeVelde', 'chrisflav', 'eric-wieser', 'github-actions', 'mistarro'] |
eric-wieser assignee:eric-wieser |
21-68868 21 days ago |
37-19762 1 month ago |
60-38464 60 days |
24379 |
chrisflav author:chrisflav |
feat(Algebra/AlgHom): `Unique` if target is `Subsingleton` |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
32/0 |
Mathlib/Algebra/Algebra/Equiv.lean,Mathlib/Algebra/Algebra/Hom.lean |
2 |
6 |
['chrisflav', 'eric-wieser', 'github-actions'] |
nobody |
21-68649 21 days ago |
60-58849 1 month ago |
61-8385 61 days |
22714 |
pfaffelh author:pfaffelh |
feat: The finite product of semi-rings (in terms of measure theory) is a semi-ring. |
~~Move results for rings (in terms of measure theory) to a separate file; was in Semiring.lean before.~~
For `∀ i ∈ s, IsSetSemiring (C i))`, the product `s.pi '' s.pi C` is a semiring.
Prove two auxiliary lemmas in `Data.Set.Prod` needed on the way.
|
large-import
new-contributor
t-measure-probability
|
264/14 |
Mathlib/Data/Set/Pairwise/Lattice.lean,Mathlib/Data/Set/Prod.lean,Mathlib/MeasureTheory/MeasurableSpace/Pi.lean,Mathlib/MeasureTheory/PiSystem.lean,Mathlib/MeasureTheory/SetSemiring.lean,lakefile.lean |
6 |
15 |
['EtienneC30', 'Paul-Lez', 'github-actions', 'leanprover-community-bot-assistant', 'pfaffelh', 'sgouezel'] |
EtienneC30 assignee:EtienneC30 |
21-68139 21 days ago |
21-68139 21 days ago |
44-84229 44 days |
25334 |
matthewjasper author:matthewjasper |
feat(RingTheory/Flat): Add theorems relating Submodule.torsion and Module.Flat |
Co-authored-by: Kevin Buzzard
---
[](https://gitpod.io/from-referrer/)
|
FLT
new-contributor
t-algebra
label:t-algebra$ |
202/0 |
Mathlib.lean,Mathlib/Algebra/Algebra/Bilinear.lean,Mathlib/Algebra/Module/LocalizedModule/Basic.lean,Mathlib/RingTheory/Flat/TorsionFree.lean,Mathlib/RingTheory/Ideal/IsPrincipal.lean |
5 |
13 |
['alreadydone', 'erdOne', 'github-actions', 'kbuzzard'] |
nobody |
21-54444 21 days ago |
30-37741 1 month ago |
30-37739 30 days |
25586 |
JovanGerb author:JovanGerb |
chore(Order): use new ge/gt naming convention - Part 5 |
This PR renames, moves around, and deprecates theorems about `PartialOrder`s
The main changes are in `Mathlib.Order.Defs.PartialOrder` and `Mathlib.Order.Basic`.
---
[](https://gitpod.io/from-referrer/)
|
|
132/121 |
Mathlib/Algebra/ContinuedFractions/Computation/Approximations.lean,Mathlib/Algebra/Exact.lean,Mathlib/Algebra/Order/AbsoluteValue/Basic.lean,Mathlib/Algebra/Order/BigOperators/Ring/Finset.lean,Mathlib/Algebra/Order/Group/PosPart.lean,Mathlib/Algebra/Order/Group/Unbundled/Abs.lean,Mathlib/Algebra/Order/Monoid/Canonical/Defs.lean,Mathlib/Algebra/Order/Monoid/Unbundled/Basic.lean,Mathlib/Algebra/Order/Ring/Unbundled/Basic.lean,Mathlib/Algebra/Quaternion.lean,Mathlib/Analysis/Analytic/Basic.lean,Mathlib/Analysis/Calculus/Darboux.lean,Mathlib/Analysis/Convex/Gauge.lean,Mathlib/Analysis/Convex/Jensen.lean,Mathlib/Analysis/Convex/Segment.lean,Mathlib/Analysis/InnerProductSpace/Basic.lean,Mathlib/Analysis/InnerProductSpace/LinearMap.lean,Mathlib/Analysis/MeanInequalities.lean,Mathlib/Analysis/Normed/Group/Basic.lean,Mathlib/Analysis/Normed/Group/Continuity.lean,Mathlib/Analysis/Normed/Group/Quotient.lean,Mathlib/Analysis/Normed/Unbundled/RingSeminorm.lean,Mathlib/Analysis/Normed/Unbundled/SeminormFromBounded.lean,Mathlib/Analysis/NormedSpace/Multilinear/Basic.lean,Mathlib/Analysis/NormedSpace/OperatorNorm/Bilinear.lean,Mathlib/Analysis/SpecialFunctions/BinaryEntropy.lean,Mathlib/Analysis/SpecialFunctions/ContinuousFunctionalCalculus/Rpow/IntegralRepresentation.lean,Mathlib/Analysis/SpecialFunctions/Pow/Real.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Inverse.lean,Mathlib/Analysis/SpecificLimits/Normed.lean,Mathlib/Combinatorics/Additive/CauchyDavenport.lean,Mathlib/Combinatorics/Additive/Energy.lean,Mathlib/Combinatorics/Configuration.lean,Mathlib/Combinatorics/SetFamily/FourFunctions.lean,Mathlib/Combinatorics/SimpleGraph/Extremal/Basic.lean,Mathlib/Data/EReal/Operations.lean,Mathlib/Data/Finset/Card.lean,Mathlib/Data/NNReal/Defs.lean,Mathlib/Data/Nat/Find.lean,Mathlib/Data/Set/Sups.lean,Mathlib/FieldTheory/Normal/Closure.lean,Mathlib/Geometry/Euclidean/Angle/Unoriented/Basic.lean,Mathlib/GroupTheory/SpecificGroups/Alternating.lean,Mathlib/LinearAlgebra/Dimension/DivisionRing.lean,Mathlib/LinearAlgebra/FreeModule/PID.lean,Mathlib/LinearAlgebra/Ray.lean,Mathlib/MeasureTheory/Measure/MeasureSpace.lean,Mathlib/NumberTheory/NumberField/CanonicalEmbedding/ConvexBody.lean,Mathlib/NumberTheory/SumFourSquares.lean,Mathlib/Order/Basic.lean,Mathlib/Order/BoundedOrder/Basic.lean,Mathlib/Order/Cover.lean,Mathlib/Order/Defs/PartialOrder.lean,Mathlib/Order/Fin/Basic.lean,Mathlib/Order/Interval/Set/Basic.lean,Mathlib/Order/UpperLower/Closure.lean,Mathlib/RingTheory/ChainOfDivisors.lean,Mathlib/RingTheory/Filtration.lean,Mathlib/RingTheory/Regular/IsSMulRegular.lean,Mathlib/SetTheory/Ordinal/Arithmetic.lean,Mathlib/SetTheory/Ordinal/Family.lean,Mathlib/Topology/Compactness/DeltaGeneratedSpace.lean,Mathlib/Topology/Instances/ENNReal/Lemmas.lean,Mathlib/Topology/Instances/ENat.lean,Mathlib/Topology/MetricSpace/HausdorffDistance.lean,Mathlib/Topology/MetricSpace/Pseudo/Defs.lean,Mathlib/Topology/Neighborhoods.lean,Mathlib/Topology/NhdsSet.lean,Mathlib/Topology/Order.lean |
69 |
3 |
['JovanGerb', 'github-actions'] |
bryangingechen assignee:bryangingechen |
21-52585 21 days ago |
22-60077 22 days ago |
22-60060 22 days |
24823 |
eric-wieser author:eric-wieser |
refactor: add `hom` lemmas for the `MonoidalCategory` structure on `ModuleCat` |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
148/164 |
Mathlib/Algebra/Category/FGModuleCat/Basic.lean,Mathlib/Algebra/Category/ModuleCat/Adjunctions.lean,Mathlib/Algebra/Category/ModuleCat/Monoidal/Basic.lean,Mathlib/Algebra/Category/ModuleCat/Monoidal/Closed.lean,Mathlib/Algebra/Category/ModuleCat/Monoidal/Symmetric.lean,Mathlib/Algebra/Category/ModuleCat/Presheaf/Free.lean,Mathlib/Algebra/Category/ModuleCat/Presheaf/Generator.lean,Mathlib/Algebra/Category/ModuleCat/Presheaf/Monoidal.lean,Mathlib/CategoryTheory/Monoidal/Internal/Module.lean,Mathlib/RepresentationTheory/Coinvariants.lean,Mathlib/RepresentationTheory/Rep.lean |
11 |
20 |
['101damnations', 'YaelDillies', 'eric-wieser', 'github-actions', 'joelriou', 'kbuzzard', 'leanprover-community-bot-assistant'] |
101damnations assignee:101damnations |
21-47773 21 days ago |
21-47792 21 days ago |
39-43838 39 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$ |
477/61 |
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 |
8 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
21-36945 21 days ago |
21-36991 21 days ago |
44-29071 44 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 |
20-86110 20 days ago |
20-86173 20 days ago |
36-31710 36 days |
23849 |
chrisflav author:chrisflav |
feat(Data/Set): add `Set.encard_iUnion` |
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-data
maintainer-merge
|
69/0 |
Mathlib/Algebra/BigOperators/Finprod.lean,Mathlib/Data/Set/Card/Arithmetic.lean,Mathlib/Data/Set/Finite/Lattice.lean |
3 |
25 |
['YaelDillies', 'chrisflav', 'github-actions'] |
YaelDillies assignee:YaelDillies |
20-60790 20 days ago |
20-60790 20 days ago |
82-74580 82 days |
25188 |
vlad902 author:vlad902 |
feat: add lemmas about `List.scanr` |
I add basic lemmas to reason about `List.scanr`, and slightly clean-up the file and add some basic lemmas to keep the API unified with the one for `List.scanl`.
---
[](https://gitpod.io/from-referrer/)
|
t-data |
84/18 |
Mathlib/Data/List/Scan.lean |
1 |
5 |
['b-mehta', 'github-actions', 'vlad902'] |
nobody |
20-56822 20 days ago |
35-79183 1 month ago |
36-16282 36 days |
25574 |
D-Thomine author:D-Thomine |
feat(Cardinal/Finite): ENat powers and cardinality |
We define the powers of an extended natural number by another extended natural numbers in a new file `Data.Enat.Pow`. We extend `Nat.card_fun` to arbitrary types in `SetTheory.Cardinal.Finite`.
- We add a few useful instances (`Pi.nonemptyUnique`, `NoZeroDivisors ℕ∞`, `Subsingleton ℕ∞ˣ`). The latter is in an odd place (`Data.Enat.Pow`), but I did not find a file with the right imports, and did not want to blow up imports in, say, `Data.Enat.Basic`.
- This PR has significant overlap with PR #16810 by @urkud . Most of it is convergent evolution (even the names), but I lifted and tweaked the `Pow` instance from there. Overall, I wouldn't mind if we first merged Yuri's PR; it would be better for documenting code contribution, but make for a more complicated process. Another solution would be to add Yuri as an author/copyright holder to `Data.Enat.Pow` if he agrees.
---
[](https://gitpod.io/from-referrer/)
|
t-set-theory
t-data
|
177/3 |
Mathlib.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/Data/ENat/Pow.lean,Mathlib/Logic/Unique.lean,Mathlib/SetTheory/Cardinal/Finite.lean |
5 |
7 |
['D-Thomine', 'github-actions', 'sgouezel'] |
nobody |
20-46590 20 days ago |
23-21076 23 days ago |
23-24997 23 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 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
PatrickMassot assignee:PatrickMassot |
20-25799 20 days ago |
103-65585 3 months ago |
103-67478 103 days |
25650 |
vlad902 author:vlad902 |
feat(SimpleGraph): Helper lemmas for Walk.take/drop |
Contributing helper lemmas I needed when formalizing Cayley graphs. |
t-combinatorics |
24/0 |
Mathlib/Combinatorics/SimpleGraph/Walk.lean |
1 |
8 |
['Rida-Hamadani', 'github-actions', 'vlad902'] |
nobody |
19-52629 19 days ago |
19-80500 19 days ago |
20-51746 20 days |
7596 |
alreadydone author:alreadydone |
feat: covering maps from properly discontinuous actions and discrete subgroups |
---
- [x] depends on: #23236
[](https://gitpod.io/from-referrer/)
|
file-removed
t-topology
|
350/21 |
Mathlib.lean,Mathlib/Analysis/SpecialFunctions/Complex/Circle.lean,Mathlib/Topology/Algebra/ConstMulAction.lean,Mathlib/Topology/Algebra/Group/Pointwise.lean,Mathlib/Topology/Covering/AddCircle.lean,Mathlib/Topology/Covering/Basic.lean,Mathlib/Topology/Covering/Galois.lean,Mathlib/Topology/Homotopy/Lifting.lean,Mathlib/Topology/Instances/AddCircle/Defs.lean |
9 |
17 |
['ADedecker', 'alreadydone', 'digama0', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'tb65536'] |
nobody |
19-50714 19 days ago |
20-25685 20 days ago |
69-19901 69 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 |
8 |
['Parcly-Taxel', 'YaelDillies', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant'] |
nobody |
19-32324 19 days ago |
19-32343 19 days ago |
80-18066 80 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$ |
255/192 |
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/Units/Regulator.lean,Mathlib/RingTheory/Ideal/Quotient/Index.lean |
15 |
23 |
['Ruben-VandeVelde', 'TwoFX', 'YaelDillies', 'alreadydone', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'loefflerd', 'madvorak', 'mathlib4-dependent-issues-bot', 'tb65536'] |
nobody |
19-25826 19 days ago |
20-49787 20 days ago |
150-39134 150 days |
25730 |
xroblot author:xroblot |
feat(ZLattice/Covolume): add `covolume_div_covolume_eq_relindex` |
Add the following result:
Let `L₁` be a sub-`ℤ`-lattice of `L₂`. Then the index of `L₁` inside `L₂` is equal to `covolume L₁ / covolume L₂`.
---
- [x] depends on: #22940
- [x] depends on: #23759
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #22961.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/22961* |
t-algebra label:t-algebra$ |
66/3 |
Mathlib/Algebra/Module/ZLattice/Basic.lean,Mathlib/Algebra/Module/ZLattice/Covolume.lean,Mathlib/GroupTheory/Index.lean,Mathlib/LinearAlgebra/Determinant.lean |
4 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
18-79534 18 days ago |
18-80625 18 days ago |
18-80610 18 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 |
1 |
['github-actions'] |
nobody |
18-76091 18 days ago |
18-76220 18 days ago |
18-76206 18 days |
25760 |
robin-carlier author:robin-carlier |
feat(CategoryTheory/Bicategory): (2,1)-categories and `Pith` |
This PR introduces a class `IsLocallyGroupoid` on bicategories, asserting that every hom-category has an `IsGroupoid` instance.
With this definition, `IsLocallyGroupoid (LocallyDiscrete C)` is correctly inferred.
Given a bicategory `B`, we introduce a type alias `Pith B` for `B` (realized as a one-field structure), and we equip it with a `Bicategory` instance where the hom-categories are the cores of the hom-categories of `B`. We show that this bicategory is a (2,1)-category, construct an inclusion pseudo-functor from `Pith B` to `B`, and show that every pseudofunctor from a (2,1)-category to `B` factors through this inclusion.
---
We can’t fully state the fact that `(pseudofunctorToPith F).comp (inclusion F)` "is" `F` because #18254 is still not merged.
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #25150.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/25150* |
t-category-theory |
191/0 |
Mathlib.lean,Mathlib/CategoryTheory/Bicategory/LocallyGroupoid.lean |
2 |
1 |
['github-actions'] |
nobody |
18-70560 18 days ago |
18-70633 18 days ago |
18-70618 18 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 |
1 |
['github-actions'] |
nobody |
18-66869 18 days ago |
18-66934 18 days ago |
18-66919 18 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.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 |
2 |
['Parcly-Taxel', 'github-actions'] |
nobody |
18-66713 18 days ago |
18-67146 18 days ago |
18-67190 18 days |
25736 |
robin-carlier author:robin-carlier |
feat(AlgebraicTopology/SimplexCategory/GeneratorsRelations/NormalForms): Normal forms for `P_σ`s |
We prove that admissible lists indeed provide a normal form for morphisms of satisfying `P_σ`.
To this end, we introduce `standardσ`, a construction that takes a list and turn it into a composition of `σ i`s in `SimplexCategoryGenRel`. We then prove that, thangs to the fifth simplicial identity, composition on the right corresponds to simplicial insertion in the list. This gives existence of a normal form for every morphism satisfying `P_σ`.
For unicity, we introduce an auxiliary function `simplicialEvalσ : (List ℕ) → ℕ → ℕ` and show that for admissible lists, it lifts to `ℕ` the `orderHom` attached to `toSimplexCategory.map standardσ`, and that we can recover elements of the list only by looking at values of this function.
Part of a series of PR formalising that `SimplexCategoryGenRel` is equivalent to `SimplexCategory`.
---
- [x] depends on: #21744
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #21745.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/21745* |
large-import
t-topology
t-category-theory
|
253/7 |
Mathlib/AlgebraicTopology/SimplexCategory/GeneratorsRelations/NormalForms.lean |
1 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
18-66133 18 days ago |
18-75823 18 days ago |
18-75811 18 days |
25786 |
Parcly-Taxel author:Parcly-Taxel |
feat: IMO 2001 Q4 |
|
IMO |
131/4 |
Archive.lean,Archive/Imo/Imo2001Q4.lean,Mathlib/Logic/Equiv/Fin/Rotate.lean |
3 |
1 |
['github-actions'] |
nobody |
18-66132 18 days ago |
18-66200 18 days ago |
18-66185 18 days |
25790 |
Parcly-Taxel author:Parcly-Taxel |
chore: remove >6 month old material in `Deprecated` |
|
file-removed
tech debt
|
0/250 |
Mathlib.lean,Mathlib/Deprecated/Cardinal/Continuum.lean,Mathlib/Deprecated/Cardinal/Finite.lean,Mathlib/Deprecated/Cardinal/PartENat.lean,Mathlib/Deprecated/Order.lean |
5 |
1 |
['github-actions'] |
nobody |
18-65389 18 days ago |
18-65488 18 days ago |
18-65476 18 days |
25794 |
dagurtomas author:dagurtomas |
feat(CategoryTheory): localization preserves braided structure |
---
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #24485.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/24485* |
t-category-theory |
733/427 |
Mathlib.lean,Mathlib/CategoryTheory/Localization/Monoidal.lean,Mathlib/CategoryTheory/Localization/Monoidal/Basic.lean,Mathlib/CategoryTheory/Localization/Monoidal/Braided.lean,Mathlib/CategoryTheory/Monoidal/Braided/Basic.lean,Mathlib/CategoryTheory/Sites/Monoidal.lean |
6 |
1 |
['github-actions'] |
nobody |
18-64176 18 days ago |
18-64248 18 days ago |
18-64233 18 days |
25795 |
dagurtomas author:dagurtomas |
chore(Condensed): introduce an abbrev for the equivalence of light condensed sets with a category of sheaves on a small site |
---
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #24522.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/24522* |
t-condensed |
39/0 |
Mathlib.lean,Mathlib/Condensed/Light/Small.lean |
2 |
1 |
['github-actions'] |
nobody |
18-64018 18 days ago |
18-64083 18 days ago |
18-64068 18 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 |
18-54594 18 days ago |
18-61293 18 days ago |
18-61278 18 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 |
133/124 |
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/Types/Colimits.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 |
28 |
3 |
['Parcly-Taxel', 'eric-wieser', 'github-actions'] |
nobody |
18-53358 18 days ago |
18-67595 18 days ago |
18-67580 18 days |
25788 |
Parcly-Taxel author:Parcly-Taxel |
feat: number of edges in the Turán graph |
We provide two theorems, the first `card_edgeFinset_turanGraph` providing the exact number of edges and the other `card_edgeFinset_turanGraph_le` providing a (slightly) looser bound whose main advantage is its lack of integer division/modulus operations.
The bound in `card_edgeFinset_turanGraph_le` is also the bound provided in [Motzkin and Straus (1965)](https://doi.org/10.4153%2FCJM-1965-053-6). |
large-import
t-combinatorics
|
132/0 |
Mathlib/Combinatorics/SimpleGraph/Turan.lean,Mathlib/Data/Nat/ModEq.lean |
2 |
2 |
['YaelDillies', 'github-actions'] |
nobody |
18-53096 18 days ago |
18-66049 18 days ago |
18-66036 18 days |
24931 |
qawbecrdtey author:qawbecrdtey |
feat(Data/Nat/Sqrt): Added lemma `Nat.add_one_sqrt_le_of_ne_zero` |
---
This commit proves a single lemma `Nat.add_one_sqrt_le_of_ne_zero`.
```lean
lemma add_one_sqrt_le_of_ne_zero {n : ℕ} (hn : n ≠ 0) : (n + 1).sqrt ≤ n
```
[](https://gitpod.io/from-referrer/)
|
t-data
easy
|
4/0 |
Mathlib/Data/Nat/Sqrt.lean |
1 |
8 |
['Ruben-VandeVelde', 'adomani', 'eric-wieser', 'github-actions', 'kckennylau', 'qawbecrdtey'] |
nobody |
18-52455 18 days ago |
46-67967 1 month ago |
46-68024 46 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 |
18-51391 18 days ago |
19-1860 19 days ago |
19-1844 19 days |
25829 |
kbuzzard author:kbuzzard |
feat: add mulEquivHaarChar |
API for the positive real factor by which an continuous multiplicative equivalence scales a regular Haar measure on a locally compact topological group.
From FLT.
---
[](https://gitpod.io/from-referrer/)
|
t-measure-probability |
158/0 |
Mathlib.lean,Mathlib/MeasureTheory/Group/Measure.lean,Mathlib/MeasureTheory/Measure/Haar/MulEquivHaarChar.lean,Mathlib/MeasureTheory/Measure/Haar/Unique.lean |
4 |
1 |
['github-actions'] |
nobody |
18-17801 18 days ago |
18-18765 18 days ago |
18-18811 18 days |
9820 |
jjaassoonn author:jjaassoonn |
feat(RingTheory/GradedAlgebra/HomogeneousIdeal): generalize to homogeneous submodule |
The definitions, constructions and theorems in `HomogeneousIdeal.lean` are generalized to a homogeneous submodules.
So say $R$ is a ring and $M \cong \bigoplus_{i} M_i$ is an $R$-module. Then a homogeneous $R$-submodule of $M$ is an $R$-submodule $N$ such that for all $i$ and $n \in N$, $n_i \in N$. Note that this notion doesn't actually require $R$ to be graded and $M$ is a graded module. But for more interesting lemmas, we do need that $M$ is graded $R$-module. We bake the fact $R$ is graded into the definition of homogeneous submodule, otherwise, `CompleteLattice HomogeneousSubmodule` cannot find the order of synthesis (the proof depends on that $R$ is graded)
All definitions/constructions/theorems have a copy for ideals as well, this is to make sure dot notation still works.
The motivation of this generalization is graded quotient module
---
- [ ] depends on:#18728
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
516/185 |
Mathlib/Algebra/Module/GradedModule.lean,Mathlib/AlgebraicGeometry/ProjectiveSpectrum/Scheme.lean,Mathlib/AlgebraicGeometry/ProjectiveSpectrum/Topology.lean,Mathlib/RingTheory/GradedAlgebra/Homogeneous/Ideal.lean,Mathlib/RingTheory/GradedAlgebra/Homogeneous/Submodule.lean,Mathlib/RingTheory/GradedAlgebra/Radical.lean,scripts/nolints_prime_decls.txt |
7 |
2 |
['github-actions'] |
nobody |
18-12916 18 days ago |
138-10999 4 months ago |
168-62138 168 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$ |
33/13 |
Mathlib/RingTheory/HahnSeries/HEval.lean |
1 |
1 |
['github-actions'] |
nobody |
18-3418 18 days ago |
18-4291 18 days ago |
18-4276 18 days |
25818 |
xroblot author:xroblot |
feat(NumberField/CMField): All CM-extensions come from the real maximal subfield |
Main result: if `K/F` is a CM-extension then `F` is isomorphic to the maximal real subfield of `K`
---
- [x] depends on: #23760
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #23858.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/23858* |
t-number-theory |
113/6 |
Mathlib/Algebra/Field/Subfield/Basic.lean,Mathlib/FieldTheory/IntermediateField/Adjoin/Basic.lean,Mathlib/FieldTheory/IntermediateField/Basic.lean,Mathlib/LinearAlgebra/Dimension/Finrank.lean,Mathlib/NumberTheory/NumberField/CMField.lean |
5 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
17-78466 17 days ago |
18-42890 18 days ago |
18-42875 18 days |
25836 |
jt496 author:jt496 |
feat(SimpleGraph/FiveWheelLike): add the Andrásfai-Erdős-Sós theorem |
Add the Andrásfai-Erdős-Sós theorem `colorable_of_cliqueFree_lt_minDegree` which says that an `r + 1`-cliquefree graph `G` with sufficiently large minimum degree is `r`-colorable.
Co-authored-by: Lian Bremner Tattersall
---
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #25313.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/25313* |
large-import
t-combinatorics
|
307/4 |
Mathlib/Combinatorics/SimpleGraph/FiveWheelLike.lean |
1 |
1 |
['github-actions'] |
nobody |
17-67705 17 days ago |
17-68554 17 days ago |
17-68542 17 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 |
17-48358 17 days ago |
17-48358 17 days ago |
17-53493 17 days |
25680 |
kim-em author:kim-em |
chore: remove some `Nat` shortcut instances |
This PR continues the work from #24928.
Original PR: https://github.com/leanprover-community/mathlib4/pull/24928 |
|
0/9 |
Mathlib/Algebra/Ring/Divisibility/Basic.lean,Mathlib/Data/List/TakeDrop.lean,Mathlib/Data/Nat/Basic.lean |
3 |
10 |
['b-mehta', 'eric-wieser', 'github-actions', 'leanprover-bot', 'mattrobball'] |
nobody |
17-47707 17 days ago |
20-16818 20 days ago |
20-16801 20 days |
25308 |
pechersky author:pechersky |
chore(Algebra/Ring/Subring): simp tag `Subring.smul_def` |
---
[](https://gitpod.io/from-referrer/)
I found this being not-simp frustrating when talking about submodules over a valuation subring. |
t-algebra label:t-algebra$ |
21/23 |
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/Submodule.lean,Mathlib/Algebra/Ring/Subring/Basic.lean,Mathlib/Algebra/Ring/Subsemiring/Basic.lean,Mathlib/Analysis/CStarAlgebra/Basic.lean,Mathlib/LinearAlgebra/RootSystem/Irreducible.lean,Mathlib/LinearAlgebra/RootSystem/RootPositive.lean,Mathlib/LinearAlgebra/RootSystem/WeylGroup.lean,Mathlib/RingTheory/Localization/InvSubmonoid.lean,Mathlib/RingTheory/OreLocalization/Basic.lean |
14 |
2 |
['eric-wieser', 'github-actions'] |
nobody |
17-21541 17 days ago |
17-21541 17 days ago |
17-46406 17 days |
25182 |
YaelDillies author:YaelDillies |
feat: `(M →* N₁) ≃* (M →* N₂)` if `N₁ ≃* N₂` |
From Toric
---
[](https://gitpod.io/from-referrer/)
|
toric
t-algebra
label:t-algebra$ |
65/12 |
Mathlib/Algebra/Category/Grp/ForgetCorepresentable.lean,Mathlib/Algebra/Category/Grp/LargeColimits.lean,Mathlib/Algebra/Category/MonCat/ForgetCorepresentable.lean,Mathlib/Algebra/Group/Equiv/Basic.lean,Mathlib/GroupTheory/FiniteAbelian/Duality.lean |
5 |
10 |
['YaelDillies', 'eric-wieser', 'github-actions'] |
nobody |
16-62742 16 days ago |
35-72066 1 month ago |
36-62706 36 days |
25856 |
MichaelStollBayreuth author:MichaelStollBayreuth |
perf(Data.Real.Sqrt): make Real.sqrt irreducible |
We try to see what happens if we make Real.sqrt irreducible.
There are cases where this makes unification very significantly faster, compare [#mathlib4 > Coercion triggers timeout @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Coercion.20triggers.20timeout/near/517177117).
(Migrated manually from #24752)
---
[](https://gitpod.io/from-referrer/)
|
migrated-from-branch
t-data
|
1/0 |
Mathlib/Data/Real/Sqrt.lean |
1 |
1 |
['github-actions'] |
nobody |
16-57238 16 days ago |
16-57238 16 days ago |
16-60944 16 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 |
49/14 |
Mathlib/Data/Nat/Digits.lean |
1 |
1 |
['github-actions'] |
nobody |
16-30075 16 days ago |
16-46991 16 days ago |
16-47038 16 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 |
10 |
['Parcly-Taxel', 'eric-wieser', 'github-actions'] |
nobody |
15-74574 15 days ago |
18-69420 18 days ago |
18-69405 18 days |
25851 |
kmill author:kmill |
feat: improve quality of proofs generated by `congr(...)`, add caching, add support for overapplied functions |
This PR makes the following improvements to the `congr(...)` term elaborator:
- It now uses `congr`/`congrFun` as much as possible instead of creating giant HEq-based congruence proofs.
- It now looks for common prefixes for applications, to skip unnecessary work proving that these parts of an application are equal.
- Intermediate results are cached.
- Overapplied functions are now supported.
An overapplied function is a function with more arguments than the arity of the function itself. For example, in `id id 2` the first `id is overapplied. The return type is conditionally a pi type depending on the values of the arguments.
Fixes Jz Pan's issue reported [on Zulip](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Strange.20error.20on.20.60congr.60.20macro/near/523998660).
Modifies a couple uses of `congr(...)` in `SimplicialSet.NerveAdjunction` to take more advantage of it.
---
[](https://gitpod.io/from-referrer/)
|
t-meta |
291/140 |
Mathlib/AlgebraicTopology/SimplicialSet/NerveAdjunction.lean,Mathlib/Tactic/TermCongr.lean,MathlibTest/TermCongr.lean |
3 |
15 |
['acmepjz', 'eric-wieser', 'github-actions', 'grunweg', 'kmill'] |
nobody |
15-73707 15 days ago |
17-17553 17 days ago |
17-17536 17 days |
25899 |
pfaffelh author:pfaffelh |
feat(Topology/Compactness/CompactSystem): introduce compact Systems |
A compact system is a set systems with the property that, whenever a countable intersections of sets in the set system is empty, there is a finite subset of sets with empty intersection. These are needed e.g. in measure theory if one wants to show sigma-additivity of a set function on a ring.
* Main result: The set of sets which are either compact and closed, or `univ`, is a compact system.
* Introduce `Dissipate s x := ⋂ y ≤ x, s y` (Data/Set/Dissipate), which is parallel to Data/Set/Accumulate.
Co-authored-by: Rémy Degenne remydegenne@gmail.com
---
*This PR continues the work from #24541.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/24541* |
|
453/2 |
Mathlib.lean,Mathlib/Data/Set/Accumulate.lean,Mathlib/Data/Set/Dissipate.lean,Mathlib/MeasureTheory/PiSystem.lean,Mathlib/Topology/Compactness/CompactSystem.lean |
5 |
1 |
['github-actions'] |
nobody |
15-60103 15 days ago |
15-60171 15 days ago |
15-60154 15 days |
25587 |
YaelDillies author:YaelDillies |
refactor: make `Rel` less see-through |
There is tension throughout the library between considering relations between `α` and `β` simply as `α → β → Prop`, or as a bundled object `Rel α β` with dedicated operations and API.
The former approach is used almost everywhere as it is very lightweight and has arguably native support from core Lean features, but it cracks at the seams whenever one starts talking about operations on relations. For example:
* composition of relations `R : α → β → Prop`, `S : β → γ → Prop` is the unwieldy `Relation.Comp R S := fun a c ↦ ∃ b, R a b ∧ S b c`
* map of a relation `R : α → β → Prop`, under `f : α → γ`, `g : β → δ` is the monstruous `Relation.map R f g := fun c d ↦ ∃ a b, r a b ∧ f a = c ∧ g b = d`.
The latter approach is embodied by the existing type `Rel α β`, with dedicated notation like `○` for composition. It makes it much easier to reason about operations relations, but currently its API suffers from the leakage of its definition as
```
def Rel (α β : Type*) := α → β → Prop
```
The fact that `Rel` isn't an `abbrev` confuses automation. But simply making it an `abbrev` would kill the point of having a separate less see-through type to perform relation operations on.
A final point, and the original motivation for this refactor, is that uniform spaces need a theory of relations on a type `α` as elements of `Set (α × α)`. This cannot be worked around, since `Set (α × α)` is the type of elements of a filter on `α × α`. This theory is already developed in `Topology.UniformSpace.Defs`, and duplicates the existing `Rel` material.
This PR is a proposal to refactor `Rel` to be less see-through by redefining it as
```
abbrev Rel (α β : Type*) := Set (α × β)
```
This has several advantages:
* The use of `α × β` means that one can't abuse the defeq of `Rel α β` with the function type `α → β → Prop`.
* Instead, we get to provide an explicit notation `a ~[R] b` that very closely follows the paper convention `a ~R b` of using relations as infixes. This notation is scoped to the `Rel` namespace.
* The use of `Set` is an extra layer of indirection to avoid automation confusing `Rel α β` with `α × β → Prop`.
* It can directly be used in the theory of uniform spaces because of the syntactic equality between `Rel α α` and `Set (α × α)`.
* A relation can still be defined from an explicit function `α → β → Prop`, with nice notation: What was previously `fun a b ↦ R a b` becomes `{(a, b) | R a b}`.
* In general, fallout is manageably small and easily fixed by inserting the `{(a, b) | R a b}` and `a ~[R] b` notations.
The benefits can be seen in places like `CategoryTheory.Category.RelCat` where automation is significantly improved, or `Combinatorics.Hall.Basic` where defeq abuse is avoided and dot notation becomes available.
---
- [x] depends on: #25593
I will add deprecations once CI passes and people agree this is a step forward.
[](https://gitpod.io/from-referrer/)
|
t-data
RFC
|
371/443 |
Mathlib/CategoryTheory/Category/RelCat.lean,Mathlib/Combinatorics/Hall/Basic.lean,Mathlib/Combinatorics/SimpleGraph/Basic.lean,Mathlib/Combinatorics/SimpleGraph/Path.lean,Mathlib/Combinatorics/SimpleGraph/Subgraph.lean,Mathlib/Data/PFun.lean,Mathlib/Data/Rel.lean,Mathlib/Order/Filter/Partial.lean,Mathlib/Order/JordanHolder.lean,Mathlib/Order/KrullDimension.lean,Mathlib/Order/Rel/GaloisConnection.lean,Mathlib/Order/RelSeries.lean,Mathlib/RingTheory/Ideal/AssociatedPrime/Finiteness.lean,Mathlib/RingTheory/Length.lean,Mathlib/RingTheory/Spectrum/Prime/LTSeries.lean |
15 |
5 |
['YaelDillies', 'eric-wieser', 'github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
15-41712 15 days ago |
15-60094 15 days ago |
15-70222 15 days |
25932 |
Garmelon author:Garmelon |
chore: remove acceptSuggestionOnEnter option |
Reverts #12749.
Discussion on zulip: [#mathlib4 > propose removing module docstring code suggestion @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/propose.20removing.20module.20docstring.20code.20suggestion/near/452477171)
---
[](https://gitpod.io/from-referrer/)
|
new-contributor |
0/1 |
.vscode/settings.json |
1 |
1 |
['github-actions'] |
nobody |
15-36073 15 days ago |
15-36144 15 days ago |
15-36136 15 days |
22078 |
Louddy author:Louddy |
feat(SkewMonoidAlgebra): multiplication and algebraic instances |
# Multiplication and Algebraic Instances
In this PR, we introduce the definition of the skewed convolution product on `SkewMonoidAlgebra k G`. Here, the product of two elements `f g : SkewMonoidAlgebra k G` is the finitely supported function whose value at `a` is the sum of `f x * (x • g y)` over all pairs `x, y` such that `x * y = a`.
We also introduce the associated algebraic instances.
## Context
This is the third part of a planned series of PRs aiming to formalise skew monoid algebras.
The PRs are split to ease the review process. The moral sum of these planned PRs is #10541.
The first and second part were #15878 and #19084.
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
new-contributor
t-algebra
label:t-algebra$ |
453/45 |
Mathlib/Algebra/SkewMonoidAlgebra/Basic.lean |
1 |
58 |
['AntoineChambert-Loir', 'Louddy', 'github-actions', 'kbuzzard'] |
nobody |
14-61499 14 days ago |
47-69480 1 month ago |
120-3609 120 days |
24254 |
Louddy author:Louddy |
feat: valuation on RatFunc which is trivial on constants |
Given a valuation `v` on `RatFunc K` that is trivial on the constants `K`, the valuation on `RatFunc.X` determines to some degree the valuation on any `p : Polynomial K`.
These are important in the context of Ostrowski's theorem for `RatFunc K`.
Note that the condition that the valuation is trivial on constants is automatically fulfilled when `K` is finite.
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$ |
93/0 |
Mathlib/FieldTheory/RatFunc/AsPolynomial.lean |
1 |
29 |
['Louddy', 'faenuccio', 'github-actions', 'mariainesdff'] |
nobody |
14-53030 14 days ago |
46-64157 1 month ago |
48-65077 48 days |
25889 |
plp127 author:plp127 |
fix(Tactic/Widget/Conv): fix various issues |
Fixes various issues with the `conv?` widget. Closes #25162.
---
[](https://gitpod.io/from-referrer/)
|
t-meta |
110/83 |
Mathlib/Tactic/Widget/Conv.lean |
1 |
1 |
['github-actions'] |
nobody |
14-52033 14 days ago |
16-6081 16 days ago |
16-6128 16 days |
25966 |
b-reinke author:b-reinke |
feat(GroupTheory/FreeGroup/ReducedWords): add theory of reduced words |
This PR continues the work from #23368.
Original PR: https://github.com/leanprover-community/mathlib4/pull/23368 |
t-algebra label:t-algebra$ |
104/0 |
Mathlib.lean,Mathlib/GroupTheory/FreeGroup/ReducedWords.lean |
2 |
2 |
['b-reinke', 'github-actions'] |
nobody |
14-45838 14 days ago |
14-45848 14 days ago |
14-45898 14 days |
25965 |
b-reinke author:b-reinke |
feat(Algebra/BigOperators/Finprod): add powerset projection lemmas |
This PR continues the work from #23926.
Original PR: https://github.com/leanprover-community/mathlib4/pull/23926 |
|
30/0 |
Mathlib/Algebra/BigOperators/Finprod.lean,Mathlib/Data/Set/Image.lean |
2 |
2 |
['b-reinke', 'github-actions'] |
joelriou assignee:joelriou |
14-41231 14 days ago |
14-46572 14 days ago |
14-46555 14 days |
25931 |
joelriou author:joelriou |
refactor(CategoryTheory): redefine triangulated subcategories using ObjectProperty |
---
This PR continues the work from #24191.
Original PR: https://github.com/leanprover-community/mathlib4/pull/24191 |
|
279/191 |
Mathlib/Algebra/Homology/DerivedCategory/Basic.lean,Mathlib/CategoryTheory/ObjectProperty/ContainsZero.lean,Mathlib/CategoryTheory/ObjectProperty/Shift.lean,Mathlib/CategoryTheory/Triangulated/HomologicalFunctor.lean,Mathlib/CategoryTheory/Triangulated/Subcategory.lean |
5 |
2 |
['github-actions', 'joelriou'] |
nobody |
14-32554 14 days ago |
15-36711 15 days ago |
15-36694 15 days |
25988 |
Multramate author:Multramate |
refactor(AlgebraicGeometry/EllipticCurve/*): replace Fin 3 with products |
This PR continues the work from #24593.
Original PR: https://github.com/leanprover-community/mathlib4/pull/24593 |
t-algebraic-geometry |
1000/1022 |
Mathlib/AlgebraicGeometry/EllipticCurve/Jacobian/Basic.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Jacobian/Formula.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Jacobian/Point.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Projective/Basic.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Projective/Formula.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Projective/Point.lean |
6 |
2 |
['Multramate', 'github-actions'] |
nobody |
14-22266 14 days ago |
14-22269 14 days ago |
14-22320 14 days |
25989 |
Multramate author:Multramate |
feat(NumberTheory/EllipticDivisibilitySequence): add elliptic nets |
This PR continues the work from #25030.
Original PR: https://github.com/leanprover-community/mathlib4/pull/25030 |
t-number-theory |
259/37 |
Mathlib/NumberTheory/EllipticDivisibilitySequence.lean |
1 |
2 |
['Multramate', 'github-actions'] |
nobody |
14-22220 14 days ago |
14-22227 14 days ago |
14-22275 14 days |
25992 |
Multramate author:Multramate |
feat(RingTheory/Ideal/Span): add pair lemmas |
This PR continues the work from #25323.
Original PR: https://github.com/leanprover-community/mathlib4/pull/25323 |
|
131/31 |
Mathlib/Algebra/Module/PID.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Affine/Point.lean,Mathlib/RingTheory/DedekindDomain/AdicValuation.lean,Mathlib/RingTheory/Ideal/Maps.lean,Mathlib/RingTheory/Ideal/Span.lean |
5 |
2 |
['Multramate', 'github-actions'] |
nobody |
14-21875 14 days ago |
14-21950 14 days ago |
14-21933 14 days |
25993 |
Multramate author:Multramate |
feat(Algebra/Group/Units/Hom): add map lemmas |
This PR continues the work from #25609.
Original PR: https://github.com/leanprover-community/mathlib4/pull/25609 |
t-algebra label:t-algebra$ |
27/10 |
Mathlib/Algebra/Group/Units/Basic.lean,Mathlib/Algebra/Group/Units/Hom.lean |
2 |
2 |
['Multramate', 'github-actions'] |
nobody |
14-21822 14 days ago |
14-21834 14 days ago |
14-21880 14 days |
25999 |
bjoernkjoshanssen author:bjoernkjoshanssen |
feat(Topology/Compactification): projective line over ℝ is homeomorphic to the one-point compactification of ℝ |
This PR continues the work from #18306.
Original PR: https://github.com/leanprover-community/mathlib4/pull/18306 |
t-topology |
920/0 |
Mathlib.lean,Mathlib/Topology/Compactification/OnePointHomeomorph.lean,Mathlib/Topology/Compactification/OnePointRealLemmas.lean |
3 |
2 |
['bjoernkjoshanssen', 'github-actions'] |
nobody |
14-2229 14 days ago |
14-2247 14 days ago |
14-2293 14 days |
24651 |
Hagb author:Hagb |
feat(RingTheory/Finiteness/Defs): span of a set is finitely generated iff generated by a finite subset |
---
- [x] depends on: #24648
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-algebra
label:t-algebra$ |
14/0 |
Mathlib/RingTheory/Finiteness/Defs.lean |
1 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
13-80774 13 days ago |
38-68768 1 month ago |
38-73319 38 days |
26013 |
tsuki8 author:tsuki8 |
feature(Data/Finset/Card,Data/Set/Finite/Basic) |
add `card_bijOn` and `finset_subset_preimage_of_finite_image`
Add `card_bijOn`: proves that for a bijection between finsets, their cardinalities are equal
Add `finset_subset_preimage_of_finite_image`: constructs a finset subset preserving image cardinality
Co-authored-by: Junyu Guo @Hagb
---
[](https://gitpod.io/from-referrer/)
|
t-data
new-contributor
|
15/0 |
Mathlib/Data/Finset/Card.lean,Mathlib/Data/Set/Finite/Basic.lean |
2 |
1 |
['github-actions'] |
nobody |
13-69077 13 days ago |
13-69133 13 days ago |
13-69186 13 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 |
13-66918 13 days ago |
13-66918 13 days ago |
13-69445 13 days |
26011 |
linesthatinterlace author:linesthatinterlace |
feat: add elementary lifts for `OneHom`, `MulHom`, `MonoidHom` and `RingHom`. |
This PR continues the work from #25264.
Original PR: https://github.com/leanprover-community/mathlib4/pull/25264 |
migrated-from-branch
t-algebra
label:t-algebra$ |
414/10 |
Mathlib/Algebra/Group/Hom/Basic.lean,Mathlib/Algebra/Group/Hom/Defs.lean,Mathlib/Algebra/Ring/Hom/Basic.lean,Mathlib/Algebra/Ring/Hom/Defs.lean |
4 |
2 |
['github-actions', 'linesthatinterlace'] |
nobody |
13-66900 13 days ago |
13-66900 13 days ago |
13-69262 13 days |
26012 |
linesthatinterlace author:linesthatinterlace |
feat: Low-level derivatives of lifts on `OneHom`, `MulHom` and `MonoidHom` |
This PR continues the work from #25290.
Original PR: https://github.com/leanprover-community/mathlib4/pull/25290 |
migrated-from-branch
t-algebra
label:t-algebra$ |
785/34 |
Mathlib/Algebra/Group/Equiv/Basic.lean,Mathlib/Algebra/Group/Hom/Basic.lean,Mathlib/Algebra/Group/Hom/Defs.lean,Mathlib/Algebra/Ring/Hom/Basic.lean,Mathlib/Algebra/Ring/Hom/Defs.lean |
5 |
2 |
['github-actions', 'linesthatinterlace'] |
nobody |
13-66893 13 days ago |
13-66893 13 days ago |
13-69209 13 days |
25327 |
YaelDillies author:YaelDillies |
feat: `F.obj M` is a commutative monoid object if `M` is |
From Toric
---
[](https://gitpod.io/from-referrer/)
|
toric |
11/3 |
Mathlib/CategoryTheory/Monoidal/CommMon_.lean,Mathlib/CategoryTheory/Monoidal/Mon_.lean |
2 |
1 |
['github-actions'] |
nobody |
13-55112 13 days ago |
30-64586 1 month ago |
30-64578 30 days |
26029 |
joelriou author:joelriou |
feat(CategoryTheory/Localization): the right derivability structure given by functorial resolutions |
This PR continues the work from #22586.
Original PR: https://github.com/leanprover-community/mathlib4/pull/22586 |
t-category-theory |
153/0 |
Mathlib.lean,Mathlib/CategoryTheory/Localization/DerivabilityStructure/OfFunctorialResolutions.lean,Mathlib/CategoryTheory/Localization/LocalizerMorphism.lean |
3 |
2 |
['github-actions', 'joelriou'] |
nobody |
13-53817 13 days ago |
13-54014 13 days ago |
13-54059 13 days |
25854 |
robin-carlier author:robin-carlier |
feat(CategoryTheory/Monoidal/Opposites): monoid objects internal to the monoidal opposite |
We construct an equivalence between monoid objects internal to a monoidal category `C`, and monoid objects internal to its monoidal opposite `Cᴹᵒᵖ`. This is done by adding `Mon_Class` and `IsMon_Hom` instance to the relevant objects, as well as by recording an explicit equivalence of categories `Mon_ C ≌ Mon_ Cᴹᵒᵖ`.
---
- [x] depends on: #25826
I made this depend on #25549 rather than making it work with the current def only to have it refactored when #25549 is merged.
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #25626.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/25626* |
t-category-theory |
112/0 |
Mathlib.lean,Mathlib/CategoryTheory/Monoidal/Opposite/Mon_.lean |
2 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
13-42112 13 days ago |
15-40055 15 days ago |
15-40040 15 days |
25767 |
robin-carlier author:robin-carlier |
feat(CategoryTheory/Monoidal/Opposite): the equivalence `Cᴹᵒᵖᴹᵒᵖ ≌ C` is monoidal |
It was left as a TODO in #10415 that the equivalence `Cᴹᵒᵖᴹᵒᵖ ≌ C` is monoidal. We clear this todo.
---
- [x] depends on: #25766
This used to be a very low-hanging fruit.
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #25628.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/25628* |
t-category-theory |
28/1 |
Mathlib/CategoryTheory/Monoidal/Opposite.lean |
1 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
13-41448 13 days ago |
15-40042 15 days ago |
15-40027 15 days |
26054 |
FMLJohn author:FMLJohn |
feat(RingTheory/GradedAlgebra/Homogeneous/Subsemiring): homogeneous subsemirings of a graded semiring |
---
[](https://gitpod.io/from-referrer/)
In this pull request, we have defined homogeneous subsemirings of `GradedRing 𝒜` where `𝒜 : ι → σ`, `SetLike σ A` and `AddSubmonoidClass σ A`.
## Main definitions
For any `R : Subsemiring A`:
* `Subsemiring.IsHomogeneous 𝒜 R`: The property that a subsemiring is closed under `GradedRing.proj`.
* `HomogeneousSubsemiring 𝒜`: The structure extending subsemirings which satisfy `Subsemiring.IsHomogeneous`. |
t-algebra label:t-algebra$ |
120/0 |
Mathlib.lean,Mathlib/RingTheory/GradedAlgebra/Homogeneous/Subsemiring.lean |
2 |
1 |
['github-actions'] |
nobody |
13-35544 13 days ago |
13-36516 13 days ago |
13-36501 13 days |
25917 |
BoltonBailey author:BoltonBailey |
docs: Add documentation arbitrarily |
This PR addresses a number of documentation linter instances.
Original PR: https://github.com/leanprover-community/mathlib4/pull/23964 |
migrated-from-branch
documentation
|
52/14 |
Mathlib/Algebra/Homology/Homotopy.lean,Mathlib/Analysis/BoxIntegral/Partition/Filter.lean,Mathlib/Control/Monad/Cont.lean,Mathlib/Data/Stream/Defs.lean,Mathlib/LinearAlgebra/AffineSpace/AffineMap.lean |
5 |
2 |
['BoltonBailey', 'github-actions'] |
nobody |
13-33874 13 days ago |
13-36039 13 days ago |
15-46068 15 days |
25919 |
BoltonBailey author:BoltonBailey |
doc: suggest !bench in `lake exe pole` |
This PR continues the work from #12561.
Original PR: https://github.com/leanprover-community/mathlib4/pull/12561 |
|
2/1 |
LongestPole/Main.lean |
1 |
2 |
['BoltonBailey', 'github-actions'] |
nobody |
13-33827 13 days ago |
13-33827 13 days ago |
15-45868 15 days |
26067 |
mapehe author:mapehe |
feat(Topology/StoneCech): exists_continuous_surjection_from_StoneCech_to_dense_range |
This lemma formalises the following version of the maximality property of the Stone–Čech compactification: If `f : α → β` is a continuous map from a topological space `α` to a Hausdorff space `β` with dense range, then there exists a continuous surjection from `StoneCech α` to `β` extending `f`. In particular, `StoneCech α` is the “largest” compact Hausdorff space into which `α` densely embeds, in the sense that any other such space is a continuous image of it.
---
[](https://gitpod.io/from-referrer/)
|
t-topology |
18/0 |
Mathlib/Topology/StoneCech.lean |
1 |
1 |
['github-actions'] |
nobody |
12-76720 12 days ago |
12-76745 12 days ago |
12-76800 12 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$ |
29/0 |
Mathlib/RingTheory/MvPolynomial/MonomialOrder.lean |
1 |
1 |
['github-actions'] |
nobody |
12-75644 12 days ago |
13-76157 13 days ago |
13-76203 13 days |
26076 |
joelriou author:joelriou |
feat(AlgebraicTopology/SimplicialSet): uniqueness of the decomposition involving non-degenerate simplices |
Any simplex `x : X _⦋n⦌` of a simplicial set can be written in a unique way as `X.map f.op y` for an epimorphism `f : ⦋n⦌ ⟶ ⦋m⦌` and a non-degenerate `m`-simplex `y`.
---
This PR continues the work from #21103.
Original PR: https://github.com/leanprover-community/mathlib4/pull/21103 |
t-topology |
118/5 |
Mathlib/AlgebraicTopology/SimplexCategory/Basic.lean,Mathlib/AlgebraicTopology/SimplicialSet/Degenerate.lean |
2 |
2 |
['github-actions', 'joelriou'] |
nobody |
12-69050 12 days ago |
12-69061 12 days ago |
12-69109 12 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 |
12-68046 12 days ago |
36-32607 1 month ago |
36-36530 36 days |
26072 |
xroblot author:xroblot |
feat(NumberField): Image of torsion modulo an ideal |
Let `I` be an integral ideal of a number field `K`. We define the morphism from the torsion of `K` to `(𝓞 K ⧸ I)ˣ` and prove that it is injective if the norm of `I` is coprime with the order of the torsion of `K`.
As a consequence, we prove that for a prime ideal `P` coprime with the order of the torsion of `K`, the norm of `P` is congruent to `1` modulo `torsionOrder K`.
|
t-number-theory |
202/1 |
Mathlib.lean,Mathlib/NumberTheory/Cyclotomic/Basic.lean,Mathlib/NumberTheory/Cyclotomic/Rat.lean,Mathlib/NumberTheory/NumberField/Ideal/Basic.lean,Mathlib/RingTheory/RootsOfUnity/PrimitiveRoots.lean |
5 |
2 |
['github-actions', 'xroblot'] |
nobody |
12-66081 12 days ago |
12-66081 12 days ago |
12-72075 12 days |
26081 |
grunweg author:grunweg |
fix/feat(migrate_to_fork.py): filter the automated summary comment as well |
[Zulip discussion](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Feedback.20on.20scripts.2Fmigrate_to_fork.2Epy/near/524149447)
---
[](https://gitpod.io/from-referrer/)
|
|
2/1 |
scripts/migrate_to_fork.py |
1 |
1 |
['github-actions'] |
nobody |
12-56154 12 days ago |
12-56234 12 days ago |
12-56217 12 days |
26080 |
grunweg author:grunweg |
feat(Tactic/Positivity): extend EReal support for numeric casts |
Extend `pos_of_isNat` and `nonneg_of_isNat` to cover monoids which are not necessarily semirings, like EReal.
[Zulip discussion](https://leanprover.zulipchat.com/#narrow/channel/113488-general/topic/.22Missing.20Tactics.22.20list/near/519660424)
---
Original PR: https://github.com/leanprover-community/mathlib4/pull/25094 |
t-meta |
76/36 |
Mathlib/Tactic/Positivity/Core.lean,MathlibTest/positivity.lean |
2 |
3 |
['YaelDillies', 'github-actions', 'grunweg'] |
nobody |
12-54256 12 days ago |
12-56812 12 days ago |
12-56906 12 days |
26099 |
grunweg author:grunweg |
feat: add IsEmbedding.sumElim_of_separatingNhds |
Characterise when the Sum.elim of two inducing maps resp. embeddings is an embedding,
and deduce that the ranges of the two maps lying in separated neighbourhoods suffices.
This is used in my bordism theory project.
Co-authored by: @plp127
---
This PR was manually re-created (and migrated to a fork at the same time) from #22137, since that seemed easiest.
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-topology
|
115/0 |
Mathlib/Data/Sum/Basic.lean,Mathlib/Topology/Constructions/SumProd.lean |
2 |
1 |
['github-actions'] |
nobody |
12-49950 12 days ago |
12-50010 12 days ago |
12-50003 12 days |
25762 |
robin-carlier author:robin-carlier |
refactor(CategoryTheory/Monoidal/Mod_): refactor `Mod_` using `MonoidalLeftAction` |
Generalize the definition of `CategoryTheory.Monoidal.Mod_Class` and `CategoryTheory.Monoidal.Mod_` to modules in `D` over a monoid object in `C`, where `C` acts monoidally on `D`.
At the same time, we refactor `Mod_` in a way similar to the one `Mon_` has been refactored in #24646. i.e we favor `Mod_Class` in the definition and `Mod_`, and introduce a Prop-class `IsMod_Hom` to define morphisms of modules.
---
- [x] depends on: #25761
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #25545.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/25545* |
t-category-theory |
203/113 |
Mathlib/CategoryTheory/Monoidal/Cartesian/Mod_.lean,Mathlib/CategoryTheory/Monoidal/Mod_.lean |
2 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
12-48951 12 days ago |
12-48951 12 days ago |
1-18084 1 day |
25365 |
YaelDillies author:YaelDillies |
feat: `CommAlgCat` is cocartesian-monoidal |
Construct the cocartesian-monoidal category structure on `CommAlgCat R` explicitly from the tensor product.
From Toric
Co-authored-by: Andrew Yang
Co-authored-by: Michał Mrugała
Co-authored-by: Christian Merten
---
[](https://gitpod.io/from-referrer/)
|
toric
t-algebra
label:t-algebra$ |
116/5 |
Mathlib.lean,Mathlib/Algebra/Category/CommAlgCat/Basic.lean,Mathlib/Algebra/Category/CommAlgCat/Monoidal.lean |
3 |
52 |
['YaelDillies', 'erdOne', 'github-actions', 'robin-carlier'] |
nobody |
12-46762 12 days ago |
28-57095 28 days ago |
28-58247 28 days |
26122 |
chrisflav author:chrisflav |
refactor(CategoryTheory/CoproductDisjoint): generalize to indexed coproducts |
We replace the currently existing `CoproductDisjoint` by a predicate for a family of objects, indicating that the pairwise
pullbacks are disjoint and the coproduct inclusions are monomorphisms.
The old predicate is recovered as `BinaryCoproductDisjoint` as an `abbrev`.
We also replace `CoproductsDisjoint` by `CoproductsOfShapeDisjoint` and `BinaryCoproductsDisjoint`. We postpone
the TODO to show that if binary coproducts are disjoint and suitable coproducts exist, then all coproducts of suitable shape are disjoint.
Note that `CoproductDisjoint` changed its meaning, so no deprecation can be added. This should be fine, since it is a leaf file that is hopefully not much used downstream.
Zulip discussion: https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/.60MonoCoprod.60.20and.20.60DisjointCoproduct.60/with/524752624
---
[](https://gitpod.io/from-referrer/)
|
t-category-theory |
198/89 |
Mathlib/CategoryTheory/Limits/Shapes/DisjointCoproduct.lean |
1 |
1 |
['github-actions'] |
nobody |
12-28336 12 days ago |
12-29617 12 days ago |
12-29601 12 days |
25949 |
themathqueen author:themathqueen |
feat(LinearAlgebra/Basis/MulOpposite): basis of an opposite space |
This adds the definition of `Basis.mulOpposite` and shows finite-dimensionality and freeness of `Hᵐᵒᵖ`.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-algebra
label:t-algebra$ |
48/0 |
Mathlib.lean,Mathlib/LinearAlgebra/Basis/MulOpposite.lean |
2 |
1 |
['github-actions'] |
nobody |
12-27526 12 days ago |
14-67835 14 days ago |
14-67881 14 days |
25874 |
themathqueen author:themathqueen |
feat(LinearAlgebra/InvariantSubmodule): invariant submodules |
Defining and proving some lemmas on invariant submodules.
This is a (2-year late) port from leanprover-community/mathlib3#18289.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-algebra
label:t-algebra$ |
176/0 |
Mathlib.lean,Mathlib/Algebra/Group/Commute/Units.lean,Mathlib/LinearAlgebra/GeneralLinearGroup.lean,Mathlib/LinearAlgebra/InvariantSubmodule.lean,Mathlib/LinearAlgebra/Projection.lean |
5 |
1 |
['github-actions'] |
nobody |
12-26440 12 days ago |
16-40066 16 days ago |
16-40113 16 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 |
12-23717 12 days ago |
16-55516 16 days ago |
16-55562 16 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 |
1 |
['b-mehta', 'github-actions'] |
nobody |
11-67805 11 days ago |
12-44464 12 days ago |
12-44517 12 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/)
|
new-contributor
t-dynamics
|
44/0 |
Mathlib.lean,Mathlib/Dynamics/BirkhoffSum/QuasiMeasurePreserving.lean |
2 |
10 |
['github-actions', 'oliver-butterley', 'sgouezel'] |
nobody |
11-67649 11 days ago |
12-71157 12 days ago |
12-71201 12 days |
24998 |
YaelDillies author:YaelDillies |
chore(Algebra/Notation): separate very basic lemmas about `Set.indicator` and `Pi.single` |
The very basic lemmas go under `Algebra.Notation` and do not import `Monoid`.
This is useful to disentangle `Finsupp` results downstream.
---
- [x] depends on: #25040
[](https://gitpod.io/from-referrer/)
|
file-removed |
720/641 |
Mathlib.lean,Mathlib/Algebra/BigOperators/Finprod.lean,Mathlib/Algebra/BigOperators/Group/Finset/Lemmas.lean,Mathlib/Algebra/BigOperators/GroupWithZero/Finset.lean,Mathlib/Algebra/BigOperators/Pi.lean,Mathlib/Algebra/Divisibility/Prod.lean,Mathlib/Algebra/Group/End.lean,Mathlib/Algebra/Group/Equiv/TypeTags.lean,Mathlib/Algebra/Group/Fin/Tuple.lean,Mathlib/Algebra/Group/Finsupp.lean,Mathlib/Algebra/Group/Hom/Defs.lean,Mathlib/Algebra/Group/Indicator.lean,Mathlib/Algebra/Group/Nat/Hom.lean,Mathlib/Algebra/Group/NatPowAssoc.lean,Mathlib/Algebra/Group/Pi/Basic.lean,Mathlib/Algebra/Group/Pointwise/Set/Scalar.lean,Mathlib/Algebra/Group/Prod.lean,Mathlib/Algebra/Group/Support.lean,Mathlib/Algebra/Group/TypeTags/Basic.lean,Mathlib/Algebra/GroupWithZero/Action/Defs.lean,Mathlib/Algebra/GroupWithZero/Indicator.lean,Mathlib/Algebra/Homology/Additive.lean,Mathlib/Algebra/Module/Basic.lean,Mathlib/Algebra/Notation/FiniteSupport.lean,Mathlib/Algebra/Notation/Indicator.lean,Mathlib/Algebra/Notation/Pi/Basic.lean,Mathlib/Algebra/Notation/Pi/Defs.lean,Mathlib/Algebra/Notation/Support.lean,Mathlib/Algebra/Order/Field/Pi.lean,Mathlib/Algebra/Order/Group/Unbundled/Abs.lean,Mathlib/Algebra/Order/GroupWithZero/Unbundled/Basic.lean,Mathlib/Algebra/Order/Sub/Prod.lean,Mathlib/Algebra/Order/Sum.lean,Mathlib/Algebra/Ring/CharZero.lean,Mathlib/Algebra/Ring/Hom/Defs.lean,Mathlib/CategoryTheory/Limits/Shapes/ZeroMorphisms.lean,Mathlib/Combinatorics/Additive/Dissociation.lean,Mathlib/Combinatorics/SimpleGraph/Bipartite.lean,Mathlib/Data/Finsupp/Basic.lean,Mathlib/Data/Finsupp/Defs.lean,Mathlib/Data/Finsupp/Single.lean,Mathlib/Data/Int/CharZero.lean,Mathlib/Data/Set/Pointwise/Support.lean,Mathlib/GroupTheory/FreeGroup/Basic.lean,Mathlib/MeasureTheory/MeasurableSpace/Basic.lean,Mathlib/Order/Filter/Basic.lean,Mathlib/Order/Filter/EventuallyConst.lean,Mathlib/Order/Interval/Set/Pi.lean,Mathlib/RingTheory/HahnSeries/Addition.lean,Mathlib/RingTheory/HahnSeries/Basic.lean,Mathlib/Topology/Algebra/Indicator.lean,Mathlib/Topology/IndicatorConstPointwise.lean,Mathlib/Topology/LocallyConstant/Basic.lean,Mathlib/Topology/LocallyFinsupp.lean,Mathlib/Topology/Separation/Basic.lean,Mathlib/Topology/Separation/DisjointCover.lean |
56 |
11 |
['YaelDillies', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
11-67612 11 days ago |
11-75248 11 days ago |
35-46664 35 days |
26141 |
kebekus author:kebekus |
feat: compute trailing coefficients of factorized rational functions |
This PR continues the work from #25523.
Original PR: https://github.com/leanprover-community/mathlib4/pull/25523 |
t-analysis |
180/3 |
Mathlib/Analysis/Meromorphic/FactorizedRational.lean,Mathlib/Analysis/Meromorphic/TrailingCoefficient.lean |
2 |
3 |
['github-actions', 'kebekus'] |
nobody |
11-64234 11 days ago |
11-64298 11 days ago |
11-64786 11 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 anyrthing about fields.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
708/638 |
Archive/Imo/Imo1982Q3.lean,Archive/Imo/Imo2013Q5.lean,Archive/Wiedijk100Theorems/PerfectNumbers.lean,Counterexamples/ZeroDivisorsInAddMonoidAlgebras.lean,Mathlib.lean,Mathlib/Algebra/Field/GeomSum.lean,Mathlib/Algebra/GeomSum.lean,Mathlib/Algebra/Order/CauSeq/BigOperators.lean,Mathlib/Algebra/Order/Field/GeomSum.lean,Mathlib/Algebra/Order/Ring/GeomSum.lean,Mathlib/Algebra/Ring/GeomSum.lean,Mathlib/Analysis/Polynomial/CauchyBound.lean,Mathlib/Analysis/SpecificLimits/Basic.lean,Mathlib/Analysis/SpecificLimits/FloorPow.lean,Mathlib/Combinatorics/Colex.lean,Mathlib/Combinatorics/SetFamily/KruskalKatona.lean,Mathlib/Data/Nat/Multiplicity.lean,Mathlib/LinearAlgebra/Projectivization/Cardinality.lean,Mathlib/LinearAlgebra/Vandermonde.lean,Mathlib/NumberTheory/Basic.lean,Mathlib/NumberTheory/FactorisationProperties.lean,Mathlib/NumberTheory/MulChar/Basic.lean,Mathlib/NumberTheory/Multiplicity.lean,Mathlib/RingTheory/AdicCompletion/Basic.lean,Mathlib/RingTheory/Ideal/Quotient/Index.lean,Mathlib/RingTheory/Idempotents.lean,Mathlib/RingTheory/IntegralDomain.lean,Mathlib/RingTheory/Nilpotent/Basic.lean,Mathlib/RingTheory/Polynomial/Basic.lean,Mathlib/Tactic/NormNum/Irrational.lean |
30 |
1 |
['github-actions'] |
nobody |
11-62555 11 days ago |
11-62555 11 days ago |
11-62550 11 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 |
11-57027 11 days ago |
11-57027 11 days ago |
11-57087 11 days |
26137 |
xroblot author:xroblot |
feat(NumberField): specialized version of Kummer Dedekind for the splitting of prime numbers (part 1) |
First part of the Kummer-Dedekind isomorphism for the splitting of rational prime numbers in number fields.
We define the `exponent` of an algebraic integer `θ` and define the isomorphism between `(ℤ / pℤ)[X] / (minpoly θ)` and `𝓞 K / p(𝓞 K)` for primes `p` which doesn't divide the exponent of `θ`.
---
[](https://gitpod.io/from-referrer/)
|
t-number-theory |
133/0 |
Mathlib.lean,Mathlib/NumberTheory/NumberField/Ideal/KummerDedekind.lean,Mathlib/Order/Atoms.lean,Mathlib/RingTheory/Ideal/Span.lean |
4 |
1 |
['github-actions'] |
nobody |
11-55528 11 days ago |
11-55528 11 days ago |
11-74282 11 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 |
11-52629 11 days ago |
11-52790 11 days ago |
11-52844 11 days |
26159 |
upobir author:upobir |
feat(Algebra/QuadraticDiscriminant): Adding inequalities on quadratic from inequalities on discriminant |
This PR continues the work from #24517.
Original PR: https://github.com/leanprover-community/mathlib4/pull/24517 |
t-algebra label:t-algebra$ |
35/0 |
Mathlib/Algebra/QuadraticDiscriminant.lean |
1 |
3 |
['github-actions', 'upobir'] |
nobody |
11-51335 11 days ago |
11-51771 11 days ago |
11-51816 11 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
|
99/32 |
Mathlib/Analysis/Convex/Cone/Basic.lean,Mathlib/Geometry/Convex/Cone/Basic.lean |
2 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
11-50716 11 days ago |
11-65141 11 days ago |
11-65814 11 days |
25002 |
YaelDillies author:YaelDillies |
chore(Finsupp): move order properties under `Order` |
---
[](https://gitpod.io/from-referrer/)
|
large-import |
357/323 |
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 |
6 |
['github-actions', 'leanprover-community-bot-assistant'] |
nobody |
11-49962 11 days ago |
11-61538 11 days ago |
11-62395 11 days |
24149 |
YaelDillies author:YaelDillies |
refactor(Convex/Cone): streamline duality |
The current library on cones is very centered around normed and Hilbert spaces.
This is inconvenient for us in Toric where we have two spaces $M$, and $N$ that are non-canonically isomorphic to $ℐ R^n$ (for the same $n$). Although we could identify $M$ and $N$ with $ℐ R^n$ and get an inner product on $M = N = ℐ R^n$ this way, we would lose the contravariance (resp. covariance) of $M$ (resp. $N$) in the group scheme that indexes them.
We would instead like to have results that apply to perfect pairings $p : M → N → ℐ R$ out of the box.
Not all the theory can be generalised, of course. So, in terms of file structure, we need to draw the line somewhere. We propose to draw it at the import of `NormedAddCommGroup`, as this is the time where the scalars suddenly get fixed to the reals, instead of an arbitrary ordered ring. This line passes through individual files, which therefore need to be split.
We operate this separation by moving the cone content that doesn't require a norm under a new folder `Geometry.Convex.Cone`. The content that does require it stays in `Analysis.Convex.Cone`. A similar operation could be performed for the rest of the `Analysis.Convex`, but it seems wiser to do so simultaneously with the convexity refactor.
Changes performed include:
* Renaming the variable `𝕜` to `R` when it is merely a ring
* Splitting files according to normless normful parts
* Completing the existing APIs
* Redefining `ProperCone R M` as an `abbrev` for `ClosedSubmodule R≥0 M`, similarly to how `PointedCone R M` is an `abbrev` for `Submodule R≥0 M`.
* Replacing the three dual cones definitions we have:
* `Set.innerDualCone : Set H → ConvexCone ℝ H`
* `PointedCone.dual : PointedCone ℝ H → PointedCone ℝ H`
* `ProperCone.dual : ProperCone ℝ H → ProperCone ℝ H`
by three new ones:
* `PointedCone.dual : Set M → PointedCone R N` for a bilinear pairing `p : M →ₗ[R] N →ₗ[R] R`
* `ProperCone.dual : Set M → ProperCone R N` for a continuous perfect pairing `p : M →ₗ[R] N →ₗ[R] R`
* `ProperCone.innerDual : Set H → ProperCone ℝ H` for an inner product space `H`
From Toric
---
- [x] depends on: #24229
- [x] depends on: #24230
- [x] depends on: #24231
- [x] depends on: #24232
- [x] depends on: #24233
- [x] depends on: #24234
- [x] depends on: #24235
- [x] depends on: #24236
- [x] depends on: #24237
- [x] depends on: #24304
- [x] depends on: #25204
- [x] depends on: #25251
- [x] depends on: #25252
[](https://gitpod.io/from-referrer/)
|
toric
t-analysis
|
395/206 |
Mathlib.lean,Mathlib/Analysis/Convex/Cone/Basic.lean,Mathlib/Analysis/Convex/Cone/Dual.lean,Mathlib/Analysis/Convex/Cone/InnerDual.lean,Mathlib/Geometry/Convex/Cone/Dual.lean,Mathlib/Geometry/Convex/Cone/README.md |
6 |
14 |
['YaelDillies', 'github-actions', 'justus-springer', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
11-49833 11 days ago |
11-50958 11 days ago |
13-47883 13 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 |
125/4 |
Mathlib/NumberTheory/Divisors.lean |
1 |
2 |
['github-actions', 'upobir'] |
nobody |
11-46086 11 days ago |
11-52123 11 days ago |
11-52168 11 days |
26152 |
ADedecker author:ADedecker |
feat: some lemmas about pointwise actions of units on filters and uniformities |
This PR continues the work from #21265.
Original PR: https://github.com/leanprover-community/mathlib4/pull/21265 |
|
49/0 |
Mathlib/Order/Filter/Pointwise.lean,Mathlib/Topology/Algebra/UniformMulAction.lean |
2 |
2 |
['ADedecker', 'github-actions'] |
nobody |
11-32299 11 days ago |
11-57403 11 days ago |
11-57386 11 days |
26170 |
linesthatinterlace author:linesthatinterlace |
feat: Add definition of `symmEquiv` |
Ad an equivalence version of `Equiv.symm` and similar operations.
---
[](https://gitpod.io/from-referrer/)
|
|
19/0 |
Mathlib/Algebra/Group/Equiv/Defs.lean,Mathlib/Algebra/Module/Equiv/Defs.lean,Mathlib/Logic/Equiv/Defs.lean |
3 |
3 |
['github-actions', 'plp127'] |
nobody |
11-29946 11 days ago |
11-48037 11 days ago |
11-48020 11 days |
26156 |
oliver-butterley author:oliver-butterley |
feat(MeasureTheory.VectorMeasure) : add a definition of total variation for VectorMeasure |
This PR adds variation for any `VectorMeasure` using a supremum definition. Currently mathlib has `TotalVariation` defined for a signed measure using the Hahn-Jordan decomposition, but this doesn't generalise.
Motivation: generally this is an important concept but specifically as a step for proving RMK in the complex case which in turn is a step to prove the spectral theorem.
Co-authored-by: @yoh-tanimoto
This PR was migrated from #25442. PR divided into smaller pieces, this is just the definition without additional lemmas. PRs adding further results related to variation are:
* #26160
* #26165
* #26168 (shows that for `SignedMeasures` the two definitions of variation coincide)
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-measure-probability
|
354/0 |
Mathlib.lean,Mathlib/MeasureTheory/VectorMeasure/Variation/Defs.lean |
2 |
1 |
['github-actions'] |
nobody |
10-73097 10 days ago |
11-54114 11 days ago |
11-54164 11 days |
26160 |
oliver-butterley author:oliver-butterley |
feat(MeasureTheory.VectorMeasure): add several lemmas which characterize variation |
Add the following lemmas concerning variation of a VectorMeasure:
* `norm_measure_le_variation`: `‖μ E‖ₑ ≤ variation μ E`.
* `variation_neg`: `(-μ).variation = μ.variation`.
* `variation_zero`: `(0 : VectorMeasure X V).variation = 0`.
* `absolutelyContinuous`
Co-authored-by: @yoh-tanimoto
Depends on
* #26156
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-measure-probability
|
432/0 |
Mathlib.lean,Mathlib/MeasureTheory/VectorMeasure/Variation/Defs.lean,Mathlib/MeasureTheory/VectorMeasure/Variation/Lemmas.lean |
3 |
1 |
['github-actions'] |
nobody |
10-73041 10 days ago |
11-51696 11 days ago |
11-51748 11 days |
26165 |
oliver-butterley author:oliver-butterley |
feat(MeasureTheory.VectorMeasure): add lemma which shows that variation of a `ℝ≥0∞` VectorMeasure is equal to itself |
Add a lemma for the variation of a VectorMeasure which tells that if `μ` is `VectorMeasure X ℝ≥0∞` then `variation μ = μ`.
Co-authored-by: @yoh-tanimoto
Depends on
* #26160
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-measure-probability
|
467/0 |
Mathlib.lean,Mathlib/MeasureTheory/VectorMeasure/Variation/Defs.lean,Mathlib/MeasureTheory/VectorMeasure/Variation/Lemmas.lean |
3 |
1 |
['github-actions'] |
nobody |
10-73020 10 days ago |
11-49092 11 days ago |
11-49139 11 days |
26168 |
oliver-butterley author:oliver-butterley |
feat(MeasureTheory.VectorMeasure) : variation defined as a supremum is equal to variation defined using the Hahn-Jordan decomposition. |
Add `signedMeasure_totalVariation_eq`: if `μ` is a `SignedMeasure` then variation defined as a supremum is equal to variation defined using the Hahn-Jordan decomposition.
Co-authored-by: @yoh-tanimoto
Depends on:
* #26165
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-measure-probability
|
680/0 |
Mathlib.lean,Mathlib/MeasureTheory/VectorMeasure/Variation/Defs.lean,Mathlib/MeasureTheory/VectorMeasure/Variation/Equiv.lean,Mathlib/MeasureTheory/VectorMeasure/Variation/Lemmas.lean |
4 |
1 |
['github-actions'] |
nobody |
10-73006 10 days ago |
11-48230 11 days ago |
11-48278 11 days |
25754 |
robin-carlier author:robin-carlier |
feat(CategoryTheory/Monoidal/ExternalProduct): external product of left Kan extended functors |
Given a functor `H' : D' ⥤ V` to a monoidal category that is pointwise left Kan extended along `L : D ⥤ D'`, we show that for a functor `K : E ⥤ V` and under suitable preservations of colimits by the tensor product of `V`, the functor `H' ⊠ K : D' × E ⥤ V` is pointwise left Kan extended along `L.prod (𝟭 E)`. We show a similar statement for the functor `K ⊠ H'`.
This property is crucial for proving properties of Day convolutions of functors from a monoidal category to `V`.
---
- [x] depends on: #25731
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #24989.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/24989* |
t-category-theory |
246/92 |
Mathlib.lean,Mathlib/CategoryTheory/Monoidal/ExternalProduct.lean,Mathlib/CategoryTheory/Monoidal/ExternalProduct/Basic.lean,Mathlib/CategoryTheory/Monoidal/ExternalProduct/KanExtension.lean |
4 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
10-71691 10 days ago |
11-83182 11 days ago |
11-83293 11 days |
26199 |
Vierkantor author:Vierkantor |
fix(Algebra): `MulMemClass.mul_mem` should not be `aesop safe` |
The `@[aesop safe apply]` attribute only applies to implications that preserve provability. So for `mul_mem (ha : a ∈ s) (hb : b ∈ s) : a * b ∈ s`, there are ways to prove `a * b ∈ s` while `b ∉ s`, such as when `s` is an ideal and `a ∈ s`.
So, instead give `MulMemClass.mul_mem` and `AddMemClass.add_mem` the unsafe attribute, and add `Ideal.mul_mem_left` and `Ideal.mul_mem_right` to the aesop with the same `unsafe` attribute. Now we can prove membership of ideals a bit more easily.
Original PR: https://github.com/leanprover-community/mathlib4/pull/24112 |
t-algebra label:t-algebra$ |
5/1 |
Mathlib/Algebra/Group/Subsemigroup/Defs.lean,Mathlib/RingTheory/Ideal/Defs.lean |
2 |
2 |
['Vierkantor', 'github-actions'] |
nobody |
10-69024 10 days ago |
10-69083 10 days ago |
10-69147 10 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 |
10-68591 10 days ago |
10-68597 10 days ago |
10-68643 10 days |
25662 |
erdOne author:erdOne |
chore: redefine `LocalizedModule` |
---
[](https://gitpod.io/from-referrer/)
|
|
197/229 |
Mathlib/Algebra/Module/LocalizedModule/Basic.lean,Mathlib/AlgebraicGeometry/Modules/Tilde.lean,Mathlib/GroupTheory/OreLocalization/Basic.lean,Mathlib/GroupTheory/OreLocalization/OreSet.lean,Mathlib/RingTheory/OreLocalization/Ring.lean,Mathlib/RingTheory/TensorProduct/Nontrivial.lean |
6 |
11 |
['erdOne', 'eric-wieser', 'github-actions', 'kckennylau', 'leanprover-bot'] |
nobody |
10-68449 10 days ago |
20-48466 20 days ago |
20-48475 20 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$ |
241/24 |
Mathlib.lean,Mathlib/Algebra/Module/Submodule/Lattice.lean,Mathlib/LinearAlgebra/Quotient/Basic.lean,Mathlib/RingTheory/Ideal/MinimalPrime/Localization.lean,Mathlib/RingTheory/KrullDimension/Module.lean,Mathlib/RingTheory/KrullDimension/Regular.lean,Mathlib/RingTheory/Nakayama.lean,Mathlib/RingTheory/Spectrum/Prime/LTSeries.lean,Mathlib/RingTheory/Support.lean |
9 |
2 |
['Thmoas-Guan', 'github-actions'] |
nobody |
10-57279 10 days ago |
10-58014 10 days ago |
10-58065 10 days |
26070 |
riccardobrasca author:riccardobrasca |
feat: add Mathlib.RingTheory.DedekindDomain.Instances |
We add a new file `Mathlib.RingTheory.DedekindDomain.Instances` containing various instances that are useful to work with the localization a prime of an extension of Dedekind domains. As a practical example we golf a tedious proof in `Mathlib.RingTheory.Ideal/Norm.RelNorm`.
---
Original PR: https://github.com/leanprover-community/mathlib4/pull/21522 |
large-import
t-algebra
t-number-theory
label:t-algebra$ |
255/73 |
Mathlib.lean,Mathlib/RingTheory/DedekindDomain/Different.lean,Mathlib/RingTheory/DedekindDomain/Instances.lean,Mathlib/RingTheory/DedekindDomain/IntegralClosure.lean,Mathlib/RingTheory/Ideal/Norm/RelNorm.lean,Mathlib/RingTheory/IntegralClosure/IntegralRestrict.lean,Mathlib/RingTheory/Localization/AtPrime.lean,Mathlib/RingTheory/Localization/Basic.lean,Mathlib/RingTheory/Localization/LocalizationLocalization.lean,Mathlib/RingTheory/RingHom/Finite.lean,Mathlib/RingTheory/Trace/Quotient.lean |
11 |
4 |
['erdOne', 'github-actions', 'riccardobrasca'] |
nobody |
10-50270 10 days ago |
12-74562 12 days ago |
12-74714 12 days |
26225 |
Raph-DG author:Raph-DG |
feat(AlgebraicGeometry): Add some minimal API for orders on schemes |
In this PR we add some minimal api for the ordering on schemes defined in #26204. We chose split these PRs because we expect there will be more discussion about this API, and having the preorder instance is useful in its own right without much added API.
- [] depends on: #26204
---
[](https://gitpod.io/from-referrer/)
|
t-algebraic-geometry |
16/0 |
Mathlib/AlgebraicGeometry/Properties.lean,Mathlib/AlgebraicGeometry/Scheme.lean |
2 |
1 |
['github-actions'] |
nobody |
10-48005 10 days ago |
10-48014 10 days ago |
10-48059 10 days |
26226 |
chrisflav author:chrisflav |
chore(AlgebraicGeometry/Limits): undeprecate `sigmaOpenCover` |
The replacement has the indexing type wrapped in `Discrete` which is inconvenient in practice.
---
[](https://gitpod.io/from-referrer/)
|
t-algebraic-geometry |
5/3 |
Mathlib/AlgebraicGeometry/Limits.lean |
1 |
1 |
['erdOne', 'github-actions'] |
nobody |
10-47201 10 days ago |
10-47489 10 days ago |
10-47474 10 days |
26220 |
linesthatinterlace author:linesthatinterlace |
fix: Removes explict `FunLike` instance for `Equiv` |
Remove explict `FunLike` instance for `Equiv`.
---
This is a somewhat experimental PR and I want to check there isn't a performance issue from doing this.
[](https://gitpod.io/from-referrer/)
|
t-logic |
24/22 |
Mathlib/Algebra/Category/AlgCat/Limits.lean,Mathlib/Algebra/Category/MonCat/Limits.lean,Mathlib/Algebra/Category/Ring/Limits.lean,Mathlib/Data/FunLike/Equiv.lean,Mathlib/Logic/Equiv/Defs.lean,Mathlib/Order/Interval/Finset/Defs.lean |
6 |
1 |
['github-actions'] |
nobody |
10-46900 10 days ago |
10-46900 10 days ago |
10-46892 10 days |
25369 |
Paul-Lez author:Paul-Lez |
feat(Order/Fin/CircularOrder): add some basic results about the circular order on Fin |
Co-authored-by: Oliver Nash
---
[](https://gitpod.io/from-referrer/)
|
t-order |
48/0 |
Mathlib.lean,Mathlib/Order/Circular.lean,Mathlib/Order/Circular/ZMod.lean |
3 |
11 |
['Paul-Lez', 'YaelDillies', 'eric-wieser', 'github-actions'] |
bryangingechen assignee:bryangingechen |
10-40220 10 days ago |
10-40220 10 days ago |
13-74213 13 days |
25941 |
erdOne author:erdOne |
feat(AlgebraicGeometry): inverse limits and schemes of finite type |
We prove the following:
Given a cofiltered diagram `D` of quasi-compact `S`-schemes with affine transition maps,
and another scheme `X` of finite type over `S`.
Then the canonical map `colim Homₛ(Dᵢ, X) ⟶ Homₛ(lim Dᵢ, X)` is injective.
Co-authored-by: Christian Merten
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebraic-geometry
|
367/3 |
Mathlib/AlgebraicGeometry/AffineTransitionLimit.lean,Mathlib/AlgebraicGeometry/Morphisms/Affine.lean,Mathlib/AlgebraicGeometry/Morphisms/FiniteType.lean,Mathlib/CategoryTheory/Limits/Constructions/Over/Connected.lean,Mathlib/CategoryTheory/Limits/Creates.lean |
5 |
15 |
['chrisflav', 'erdOne', 'github-actions'] |
nobody |
10-32824 10 days ago |
15-15542 15 days ago |
15-15603 15 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 |
10-27249 10 days ago |
11-84540 11 days ago |
11-84524 11 days |
25883 |
pfaffelh author:pfaffelh |
feat: introduce Gram matrices |
A Gram matrix has entry `⟪v i, v j⟫` at `i j : n`, where `v : n → α` is an `InnerProductSpace 𝕜 α`.
Give this notion and show that Gram matrices are positive semi-definite.
This will be used later in order to show that the covariance matrix for Brownian Motion is positive semi-definite.
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #24575.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/24575* |
migrated-from-branch
new-contributor
|
157/2 |
Mathlib.lean,Mathlib/Analysis/InnerProductSpace/GramMatrix.lean,Mathlib/MeasureTheory/Function/L2Space.lean |
3 |
8 |
['eric-wieser', 'github-actions', 'pfaffelh'] |
nobody |
10-23354 10 days ago |
16-24604 16 days ago |
16-24958 16 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 |
10-21405 10 days ago |
10-21405 10 days ago |
10-26018 10 days |
26243 |
DavidLedvinka author:DavidLedvinka |
feat(Topology): Add PairReduction.lean |
Add file PairReduction.lean which proves the theorem `pair_reduction` which is needed for the proof of the general Kolmogorov-Chentsov theorem in the Brownian Motion project.
Co-authored-by: @RemyDegenne |
t-topology |
435/0 |
Mathlib.lean,Mathlib/Topology/EMetricSpace/PairReduction.lean |
2 |
1 |
['github-actions'] |
nobody |
9-79436 9 days ago |
10-4312 10 days ago |
0-1394 23 minutes |
26258 |
kckennylau author:kckennylau |
feat(Topology): induction for sheafification |
---
I currently have binary and unary operation, which should be enough for sheaves.
[](https://gitpod.io/from-referrer/)
|
t-topology |
62/1 |
Mathlib/Topology/Sheaves/LocalPredicate.lean |
1 |
1 |
['github-actions'] |
nobody |
9-35035 9 days ago |
9-35144 9 days ago |
9-35207 9 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 |
9-32910 9 days ago |
13-14174 13 days ago |
13-14222 13 days |
26259 |
Raph-DG author:Raph-DG |
feat(Topology): Connecting different notions of locally finite |
In this PR we connect the notions of local finiteness of an indexed family of sets (as in LocallyFinite) and of a set of sets (as in Function.locallyFinsuppWithin)
---
[](https://gitpod.io/from-referrer/)
|
t-topology |
32/0 |
Mathlib/Topology/LocallyFinsupp.lean |
1 |
3 |
['Raph-DG', 'github-actions', 'kckennylau'] |
nobody |
8-72778 8 days ago |
9-34939 9 days ago |
9-34982 9 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 |
8-50023 8 days ago |
12-31359 12 days ago |
12-31411 12 days |
26247 |
vasnesterov author:vasnesterov |
perf(Topology/Metrizable): lower `IsCompletelyMetrizableSpace.MetrizableSpace` priority |
This PR continues the work from #24967.
Original PR: https://github.com/leanprover-community/mathlib4/pull/24967 |
t-topology
easy
|
3/1 |
Mathlib/Topology/Metrizable/CompletelyMetrizable.lean |
1 |
6 |
['github-actions', 'mathlib-bors', 'vasnesterov'] |
nobody |
8-49112 8 days ago |
8-49113 8 days ago |
9-69528 9 days |
25837 |
jt496 author:jt496 |
feat(Combinatorics/SimpleGraph): add homOfConnectedComponents and related results |
Given homomorphisms of each connected component of `G : SimpleGraph α` into `H : SimpleGraph β `give the corresponding `G →g H`
Hence prove that G is n - colorable iff each connected component is n - colorable.
Also prove that G is 2-colorable iff it does not contain an odd length loop (closed walk).
I wasn't sure where to put this - it probably belongs in SimpleGraph.ConcreteColorings?
---
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #24546.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/24546* |
t-combinatorics |
36/0 |
Mathlib/Combinatorics/SimpleGraph/Coloring.lean,Mathlib/Combinatorics/SimpleGraph/ConcreteColorings.lean,Mathlib/Combinatorics/SimpleGraph/Connectivity/Connected.lean |
3 |
1 |
['github-actions'] |
nobody |
8-46303 8 days ago |
17-68437 17 days ago |
17-68423 17 days |
26271 |
Raph-DG author:Raph-DG |
feat(AlgebraicGeometry): Simple lemma about existence of affine neighbourhoods |
In this PR we make a simple lemma saying there exists an affine open around any point in a scheme. This already exists in the language of open immersions, this just makes the construction of the affine open subset more convenient.
---
[](https://gitpod.io/from-referrer/)
|
t-algebraic-geometry |
6/0 |
Mathlib/AlgebraicGeometry/AffineScheme.lean |
1 |
1 |
['github-actions'] |
nobody |
8-43615 8 days ago |
8-47701 8 days ago |
8-47746 8 days |
26059 |
wwylele author:wwylele |
feat(GroupTheory/Divisible): Add rational SMul and Module |
This is part of https://github.com/leanprover-community/mathlib4/pull/25140. A torsion-free ℕ-divisible commutative group is a ℚ-module.
----
This PR continues the work from #25190.
Original PR: https://github.com/leanprover-community/mathlib4/pull/25190 |
t-algebra label:t-algebra$ |
156/0 |
Mathlib/Data/NNRat/Lemmas.lean,Mathlib/Data/Rat/Lemmas.lean,Mathlib/GroupTheory/Divisible.lean |
3 |
5 |
['eric-wieser', 'github-actions', 'wwylele'] |
nobody |
8-19964 8 days ago |
13-13705 13 days ago |
13-13727 13 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 |
7-86007 7 days ago |
7-86030 7 days ago |
8-13547 8 days |
25860 |
robin-carlier author:robin-carlier |
feat(CategoryTheory/Monoidal/Action): Action of monoidal opposites |
Given a monoidal category `C` and a category `D`, we prove that a left (resp. right) `Cᴹᵒᵖ`-action on `D` gives a right (resp. left) `C`-action on `D`. Conversely, we show that left/right `C`-actions gives right/left `Cᴹᵒᵖ`-actions.
---
- [x] depends on: #25840
[](https://gitpod.io/from-referrer/)
|
t-category-theory |
190/1 |
Mathlib.lean,Mathlib/CategoryTheory/Monoidal/Action/Basic.lean,Mathlib/CategoryTheory/Monoidal/Action/Opposites.lean |
3 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
7-75797 7 days ago |
7-75962 7 days ago |
8-29335 8 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 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
7-75517 7 days ago |
7-75517 7 days ago |
8-27367 8 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
|
149/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 |
7-67584 7 days ago |
12-31312 12 days ago |
13-7769 13 days |
26296 |
alreadydone author:alreadydone |
feat: closure of rationals in real intervals |
Show that any `OrdConnected` set of real numbers has the same closure as the set of rational numbers in it.
---
[](https://gitpod.io/from-referrer/)
|
t-topology |
23/9 |
Mathlib/Algebra/Order/Archimedean/Basic.lean,Mathlib/Topology/Instances/Real/Lemmas.lean |
2 |
1 |
['github-actions'] |
nobody |
7-63526 7 days ago |
7-63526 7 days ago |
7-64456 7 days |
25976 |
robin-carlier author:robin-carlier |
feat(CategoryTheory/Monoidal/Action): preservation of left/right actions by functors |
We introduce typeclasses `F.LaxLeftLinear C`, `F.OplaxLeftLinear C` and `F.LeftLinear C` on functors `F : D ⥤ D'` where `D` and `D` have a monoidal left action of `C`. These typeclasses bundle "compatibility" of the actions, and are analogue to `LaxMonoidal` and `OplaxMonoidal` structures on functors.
More precisely, `F.LaxLeftLinear C` bundles a"lineator" as a morphism `μₗ : c ⊙ₗ F.obj d ⟶ F.obj (c ⊙ₗ d)`, subject to naturality, associativity and unitality conditions while `F.OplaxLeftLinear C` bundles the "lineator" as a morphism `δₗ : F.obj (c ⊙ₗ d) ⟶ c ⊙ₗ F.obj d ` subject to similar conditions. `F.LeftLinear` bundles both a `LaxLeftLinear` and an `OplaxLeftLinear` structure, as well as the fact that `μₗ` is left and right inverse to `δₗ`.
The analogue typeclasses for right actions are also introduced.
---
- [x] depends on: #25840
[](https://gitpod.io/from-referrer/)
|
t-category-theory |
361/1 |
Mathlib.lean,Mathlib/CategoryTheory/Monoidal/Action/Basic.lean,Mathlib/CategoryTheory/Monoidal/Action/LinearFunctor.lean |
3 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
7-58438 7 days ago |
7-75481 7 days ago |
8-27987 8 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$ |
305/0 |
Mathlib.lean,Mathlib/RingTheory/Bialgebra/GroupLike.lean,Mathlib/RingTheory/Coalgebra/GroupLike.lean,Mathlib/RingTheory/HopfAlgebra/GroupLike.lean |
4 |
30 |
['Julian-Kuelshammer', 'Parcly-Taxel', 'YaelDillies', 'erdOne', 'eric-wieser', 'github-actions', 'leanprover-bot', 'mathlib4-dependent-issues-bot'] |
nobody |
7-56121 7 days ago |
51-23178 1 month ago |
51-24733 51 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 |
7-53397 7 days ago |
7-53407 7 days ago |
7-53452 7 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 |
5 |
['github-actions', 'loefflerd', 'sgouezel'] |
nobody |
7-52789 7 days ago |
15-39290 15 days ago |
17-70478 17 days |
26299 |
adomani author:adomani |
perf: the `commandStart` linter only acts on modified files |
Introduces an `IO.Ref` to allow the `commandStart` linter to only run on files that git considers modified with respect to `master`.
The linter is also active on files that have had some error, as these are likely being modified!
The PR should also mitigate the speed-up that the linter introduced:
[#mathlib4 > A whitespace linter @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/A.20whitespace.20linter/near/525091877)
Assuming that this goes well, a similar mechanism could be applied to several linters that do not need to run on all code, just on the modified code.
Implementation detail: the linter is currently either on or off in "whole" files. It may be also a future development to make this more granular and only run the linter on "modifed commands in modified files", but this is not currently the plan for this modification!
---
[](https://gitpod.io/from-referrer/)
|
t-linter |
48/0 |
Mathlib/Tactic/Linter/CommandStart.lean |
1 |
4 |
['adomani', 'github-actions', 'leanprover-bot'] |
nobody |
7-52722 7 days ago |
7-52722 7 days ago |
7-57355 7 days |
26189 |
tb65536 author:tb65536 |
feat(FieldTheory/Galois/Basic): Add simp-lemma for `FixedPoints.intermediateField` |
This PR adds a simp-lemma `FixedPoints.mem_intermediateField_iff` for the definition `FixedPoints.intermediateField`.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
4/0 |
Mathlib/FieldTheory/Galois/Basic.lean |
1 |
1 |
['github-actions'] |
nobody |
7-46907 7 days ago |
7-46907 7 days ago |
11-18158 11 days |
26308 |
LessnessRandomness author:LessnessRandomness |
feat(Analysis.NormedSpace): add normalized vectors |
---
Add normalized vectors to Mathlib (zero vector for zero vector, the corresponding unit vectors for nonzero vectors) |
new-contributor
t-analysis
|
65/0 |
Mathlib.lean,Mathlib/Analysis/NormedSpace/Normalized.lean |
2 |
1 |
['github-actions'] |
nobody |
7-45502 7 days ago |
7-45514 7 days ago |
7-45560 7 days |
25997 |
tb65536 author:tb65536 |
refactor(FieldTheory/Galois): Switch from `Fintype` to `Finite` |
This PR switches mathlib's Galois theory from `Fintype` to `Finite` to match the group theory library.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
59/61 |
Mathlib/FieldTheory/Galois/Basic.lean,Mathlib/FieldTheory/Galois/IsGaloisGroup.lean,Mathlib/FieldTheory/IntermediateField/Adjoin/Basic.lean,Mathlib/FieldTheory/KrullTopology.lean,Mathlib/FieldTheory/KummerExtension.lean,Mathlib/FieldTheory/PolynomialGaloisGroup.lean,Mathlib/NumberTheory/NumberField/CMField.lean,Mathlib/NumberTheory/NumberField/InfinitePlace/Ramification.lean |
8 |
1 |
['github-actions'] |
nobody |
7-44770 7 days ago |
7-44770 7 days ago |
13-51213 13 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 |
7-43867 7 days ago |
7-43868 7 days ago |
11-13470 11 days |
26316 |
alreadydone author:alreadydone |
feat(RingTheory): degree of rational function field extension |
This PR continues the work from #22966.
Original PR: https://github.com/leanprover-community/mathlib4/pull/22966 |
t-algebra label:t-algebra$ |
268/49 |
Mathlib/RingTheory/AdjoinRoot.lean,Mathlib/RingTheory/Algebraic/Basic.lean,Mathlib/RingTheory/Algebraic/Integral.lean,Mathlib/RingTheory/AlgebraicIndependent/AlgebraicClosure.lean,Mathlib/RingTheory/IntegralClosure/IsIntegralClosure/Basic.lean,Mathlib/RingTheory/TensorProduct/Basic.lean |
6 |
2 |
['alreadydone', 'github-actions'] |
riccardobrasca assignee:riccardobrasca |
7-40711 7 days ago |
7-40718 7 days ago |
7-43354 7 days |
26319 |
Vierkantor author:Vierkantor |
ci: specify leanprover-community/mathlib4 when checking out master |
This PR makes it explicit that we want to run CI against the `master` branch from `leanprover-community/mathlib4` instead of another repo.
The new mathlib4-nightly-testing repo should run CI on the nightly branches as if they are already part of the `master` branch. But when checking them out, it defaults to looking for the branch in `leanprover-community/mathlib4-nightly-testing`, which does not exist. So a simple fix is to make the upstream repo name explicit.
A potential disadvantage: it will be harder to test CI changes by opening a pull request against one's own fork. (Which is what I did to test a few CI changes before).
---
This change makes sense to me but maybe there is a better option? I don't think we want to have custom CI in the other repo, because it will get obliterated next time we do an update.
[](https://gitpod.io/from-referrer/)
|
CI |
4/0 |
.github/build.in.yml,.github/workflows/bors.yml,.github/workflows/build.yml,.github/workflows/build_fork.yml |
4 |
1 |
['github-actions'] |
nobody |
7-38762 7 days ago |
7-38831 7 days ago |
7-38815 7 days |
25283 |
Brian-Nugent author:Brian-Nugent |
feat: regular local rings |
Adds regular local rings and proves they are integral domains.
---
- [ ] depends on: #25280
- [ ] depends on: #25282
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-algebra
label:t-algebra$ |
871/0 |
.vscode/settings.json,Mathlib.lean,Mathlib/RingTheory/EmbeddingDimension.lean,Mathlib/RingTheory/LocalRingDimension.lean,Mathlib/RingTheory/RegularLocalRing.lean |
5 |
5 |
['Brian-Nugent', 'github-actions', 'mathlib4-dependent-issues-bot', 'yuanyi-350'] |
nobody |
7-24844 7 days ago |
7-84702 7 days ago |
7-85567 7 days |
26265 |
EtienneC30 author:EtienneC30 |
feat: random variables are independent iff their joint distribution is the product measure |
Also prove that random variables are independent iff any finite subfamily is independent.
---
[](https://gitpod.io/from-referrer/)
|
t-measure-probability |
109/8 |
Mathlib.lean,Mathlib/MeasureTheory/Measure/MeasureSpaceDef.lean,Mathlib/Probability/Independence/Basic.lean,Mathlib/Probability/Independence/InfinitePi.lean,Mathlib/Probability/Independence/Kernel.lean |
5 |
4 |
['EtienneC30', 'github-actions', 'sgouezel'] |
nobody |
7-24185 7 days ago |
8-69273 8 days ago |
8-69257 8 days |
26325 |
TOMILO87 author:TOMILO87 |
feat: beta distribution |
This PR continues the work from #25608.
Original PR: https://github.com/leanprover-community/mathlib4/pull/25608 |
new-contributor
t-measure-probability
|
257/0 |
Mathlib.lean,Mathlib/Probability/Distributions/Beta.lean |
2 |
2 |
['TOMILO87', 'github-actions'] |
nobody |
7-22793 7 days ago |
7-22803 7 days ago |
7-22845 7 days |
26078 |
kckennylau author:kckennylau |
feat(AlgebraicGeometry): add x, y, px, py for points on elliptic curves |
---
Split from #25218.
[](https://gitpod.io/from-referrer/)
|
t-algebraic-geometry |
44/0 |
Mathlib/AlgebraicGeometry/EllipticCurve/Affine/Point.lean |
1 |
10 |
['MichaelStollBayreuth', 'Multramate', 'acmepjz', 'github-actions', 'kckennylau'] |
nobody |
7-20301 7 days ago |
12-58807 12 days ago |
12-58853 12 days |
26330 |
Timeroot author:Timeroot |
"Junk value" test file |
This PR continues the work from #25173.
Original PR: https://github.com/leanprover-community/mathlib4/pull/25173 |
t-data |
362/2 |
Mathlib/Data/Nat/Find.lean,MathlibTest/Junk.lean |
2 |
2 |
['Timeroot', 'github-actions'] |
nobody |
7-5320 7 days ago |
7-5326 7 days ago |
7-5372 7 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 |
7-5052 7 days ago |
7-5059 7 days ago |
7-5103 7 days |
23460 |
Timeroot author:Timeroot |
feat: Definition of `Clone` |
Basics about Clones. Part of #20051
---
- [x] depends on: #23459
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
326/0 |
Mathlib.lean,Mathlib/Algebra/Clone/Basic.lean,Mathlib/Algebra/Clone/Defs.lean,Mathlib/Data/Fin/Basic.lean |
4 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
7-4501 7 days ago |
7-4503 7 days ago |
7-5796 7 days |
26331 |
Timeroot author:Timeroot |
feat(Algebra/Polynomial): Descartes' Rule of signs |
This PR continues the work from #23681.
Original PR: https://github.com/leanprover-community/mathlib4/pull/23681 |
t-algebra label:t-algebra$ |
615/3 |
Mathlib.lean,Mathlib/Algebra/Polynomial/CoeffList.lean,Mathlib/Algebra/Polynomial/Degree/Operations.lean,Mathlib/Algebra/Polynomial/EraseLead.lean,Mathlib/Algebra/Polynomial/RuleOfSigns.lean |
5 |
5 |
['Timeroot', 'adomani', 'github-actions'] |
nobody |
7-1950 7 days ago |
7-5170 7 days ago |
7-5216 7 days |
26274 |
EtienneC30 author:EtienneC30 |
feat: api for symmetric bilinear forms |
Change the definition of `BilinForm.IsSymm` to make it a structure, in order to extend it to define `ContinuousBilinForm.IsPosSemidef` in #26315.
Prove polarization identity.
Prove two lemmas about `BilinForm.toMatrix`.
---
From Brownian motion
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
88/17 |
Mathlib/LinearAlgebra/BilinearForm/Orthogonal.lean,Mathlib/LinearAlgebra/BilinearForm/Properties.lean,Mathlib/LinearAlgebra/Matrix/BilinearForm.lean,Mathlib/RingTheory/Trace/Defs.lean |
4 |
2 |
['bryangingechen', 'github-actions'] |
nobody |
6-76682 6 days ago |
6-76682 6 days ago |
7-4655 7 days |
26255 |
vasnesterov author:vasnesterov |
feat(Analysis): radius of convergence for `FormalMultilinearSeries.compContinuousLinearMap` |
- Add basic lemmas `compContinuousLinearMap_id` and `compContinuousLinearMap_comp`.
- Prove lower and upper bounds for the convergence radius of `f.compContinuousLinearMap`.
- Prove `radius_compNeg`: the convergence radii of `f(x)` and `f(-x)` are equal.
---
In this PR I had to add `set_option linter.style.longFile 1700` in `Analytic/Basic.lean`.
I split this file in the next PR: #26270.
[](https://gitpod.io/from-referrer/)
This PR continues the work from #22531.
Original PR: https://github.com/leanprover-community/mathlib4/pull/22531 |
t-analysis |
148/11 |
Mathlib/Analysis/Analytic/Basic.lean,Mathlib/Analysis/Analytic/CPolynomial.lean,Mathlib/Analysis/Analytic/Constructions.lean,Mathlib/Analysis/Calculus/FormalMultilinearSeries.lean,Mathlib/Analysis/NormedSpace/OperatorNorm/NormedSpace.lean |
5 |
11 |
['github-actions', 'grunweg', 'vasnesterov'] |
grunweg assignee:grunweg |
6-33662 6 days ago |
7-50291 7 days ago |
9-23291 9 days |
26367 |
sgouezel author:sgouezel |
chore: disable `--fail` flag in curl |
See Zulip discussion at [#mathlib4 > lake exe cache get very slow @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/lake.20exe.20cache.20get.20very.20slow/near/523788423)
This is a very big improvement for me on curl 8.13.0 (download goes from 2 hours to 5 seconds!), but I haven't tested if this has bad consequences on other curl versions.
---
[](https://gitpod.io/from-referrer/)
|
|
3/1 |
Cache/Requests.lean |
1 |
1 |
['github-actions'] |
nobody |
5-79280 5 days ago |
6-39983 6 days ago |
6-39967 6 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 |
5-69258 5 days ago |
7-43905 7 days ago |
7-43957 7 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 |
1 |
['github-actions'] |
nobody |
5-65297 5 days ago |
10-68185 10 days ago |
10-68230 10 days |
25974 |
scholzhannah author:scholzhannah |
feat(Topology/Compactness/CompactlyCoherentSpace): compact coherentification (k-ification) |
This PR defines the notion of turning an arbitrary topological space into a compactly coherent space. Compactly coherent spaces are commonly referred to as "compactly generated spaces" or "k-spaces" in the literature while the operation of turning a space into such as space is called the "k-ification". There are however three different notions that are described with this name. To disambiguate we use the names "compactly coherent space" and "compactcoherentification" here. See [this wikipedia page](https://en.wikipedia.org/wiki/Compactly_generated_space) for an explanation of these notions.
This PR continues the work from #25318.
Original PR: https://github.com/leanprover-community/mathlib4/pull/25318
Co-authored-by: Floris van Doorn |
large-import
t-topology
|
175/5 |
Mathlib/Topology/Compactness/CompactlyCoherentSpace.lean |
1 |
2 |
['github-actions', 'scholzhannah'] |
nobody |
5-65198 5 days ago |
14-30718 14 days ago |
14-30768 14 days |
26415 |
thorimur author:thorimur |
feat: basic translations between `X →o Y` and `X ⥤ Y` |
Adds basic definitions translating between `X →o Y` and `X ⥤ Y` where `X` and `Y` are regarded as `Preorder` categories.
---
[](https://gitpod.io/from-referrer/)
|
t-category-theory |
53/14 |
Mathlib/CategoryTheory/Category/Preorder.lean |
1 |
2 |
['github-actions', 'thorimur'] |
nobody |
5-14768 5 days ago |
5-14768 5 days ago |
5-15110 5 days |
26435 |
kim-em author:kim-em |
chore: testing CI updates from #26439 |
---
[](https://gitpod.io/from-referrer/)
|
t-computability |
1/0 |
Mathlib/Computability/AkraBazzi/AkraBazzi.lean |
1 |
1 |
['github-actions'] |
nobody |
4-48331 4 days ago |
4-57377 4 days ago |
4-57421 4 days |
26368 |
Whysoserioushah author:Whysoserioushah |
feat(RingTheory/TwoSidedIdeal/SpanAsSum): span of set as finsum |
Reopened after everything moved to fork.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
81/0 |
Mathlib.lean,Mathlib/RingTheory/TwoSidedIdeal/SpanAsSum.lean |
2 |
1 |
['github-actions'] |
nobody |
4-36406 4 days ago |
6-34474 6 days ago |
6-34522 6 days |
26445 |
kim-em author:kim-em |
chore: use deep clones in CI |
|
CI |
3/0 |
.github/build.in.yml |
1 |
2 |
['eric-wieser', 'github-actions'] |
nobody |
4-30482 4 days ago |
4-49323 4 days ago |
4-49367 4 days |
26354 |
vasnesterov author:vasnesterov |
feat(Tactic/Order): support `⊤`, `⊥`, and lattice operations |
Support `⊤`, `⊥`, and lattice operations in the `order` tactic.
---
- [x] depends on: #21877
[](https://gitpod.io/from-referrer/)
This PR continues the work from #21966.
Original PR: https://github.com/leanprover-community/mathlib4/pull/21966 |
large-import
t-meta
|
300/107 |
Mathlib/Tactic/Order.lean,Mathlib/Tactic/Order/CollectFacts.lean,Mathlib/Tactic/Order/Graph/Basic.lean,Mathlib/Tactic/Order/Preprocessing.lean,MathlibTest/order.lean,scripts/noshake.json |
6 |
15 |
['JovanGerb', 'github-actions', 'mathlib4-dependent-issues-bot', 'vasnesterov'] |
nobody |
4-29761 4 days ago |
6-56269 6 days ago |
6-56326 6 days |
25172 |
eric-wieser author:eric-wieser |
feat: restricting `Affine.Simplex` to an affine subspace that contains it |
Also removes a redundant `Nonempty` argument.
---
[](https://gitpod.io/from-referrer/)
|
maintainer-merge
t-euclidean-geometry
|
68/5 |
Mathlib/LinearAlgebra/AffineSpace/AffineSubspace/Basic.lean,Mathlib/LinearAlgebra/AffineSpace/Independent.lean |
2 |
11 |
['eric-wieser', 'github-actions', 'jsm28', 'ocfnash'] |
nobody |
4-29694 4 days ago |
36-56285 1 month ago |
37-10758 37 days |
26375 |
joelriou author:joelriou |
chore(CategoryTheory/Localization): fix morphisms in the category of resolutions |
This PR changes the definition of morphisms in the categories `LeftResolution` and `RightResolution` attached to morphisms of localizers. Previously, we assumed that morphisms between resolutions belonged to the given class of morphisms of the localizer, but in downstream applications, it turns out it is more convenient to remove this condition (which would anyway be automatically verified in most situations). (The literature is not very explicit about whether this condition should or should not be part of the definition.)
---
[](https://gitpod.io/from-referrer/)
|
t-category-theory |
12/27 |
Mathlib/CategoryTheory/Localization/DerivabilityStructure/Constructor.lean,Mathlib/CategoryTheory/Localization/Resolution.lean |
2 |
1 |
['github-actions'] |
nobody |
4-29490 4 days ago |
6-29417 6 days ago |
6-29402 6 days |
25937 |
101damnations author:101damnations |
feat(RepresentationTheory/GroupCohomology): add Shapiro's lemma |
Given a commutative ring `k` and a finite index subgroup `S ≤ G`, the file `RepresentationTheory/FiniteIndex.lean` defines a natural isomorphism between the functors `Ind_S^G, Coind_S^G : Rep k S ⥤ Rep k G`.
Using this isomorphism, we conclude that the `(Co)ind_S^G` and `Res(S) : Rep k G ⥤ Rep k S` are both left and right adjoint to each other, and thus that `Res(S)` is an exact functor which preserves projective objects. In particular, given a projective resolution `P` of `k` as a trivial `k`-linear `G`-representation, `Res(S)(P)` is a projective resolution of `k` as a trivial `k`-linear `S`-representation.
Since `Hom(Res(S)(P), A) ≅ Hom(P, Coind_S^G(A))` for any `S`-representation `A`, we conclude Shapiro's lemma for group cohomology: `Hⁿ(G, Coind_S^G(A)) ≅ Hⁿ(S, A)` for all `n`.
---
- [x] depends on: #25869
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
112/13 |
Mathlib.lean,Mathlib/CategoryTheory/Preadditive/Projective/Resolution.lean,Mathlib/RepresentationTheory/Coinduced.lean,Mathlib/RepresentationTheory/FiniteIndex.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/Basic.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/Shapiro.lean,Mathlib/RepresentationTheory/Induced.lean |
7 |
n/a |
['101damnations', 'github-actions', 'mathlib4-dependent-issues-bot', 'tb65536'] |
nobody |
4-29214 4 days ago |
unknown |
unknown |
26428 |
Ruben-VandeVelde author:Ruben-VandeVelde |
feat: norm_num support for Int.fract |
---
[](https://gitpod.io/from-referrer/)
|
t-data |
44/0 |
Mathlib/Data/Rat/Floor.lean,MathlibTest/norm_num_ext.lean |
2 |
5 |
['Rob23oba', 'github-actions'] |
nobody |
4-25262 4 days ago |
4-25303 4 days ago |
4-70064 4 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 |
98/120 |
Archive/Wiedijk100Theorems/AscendingDescendingSequences.lean |
1 |
12 |
['b-mehta', 'github-actions', 'grunweg'] |
nobody |
4-11591 4 days ago |
4-65217 4 days ago |
6-33757 6 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
|
134/27 |
Mathlib/Algebra/Category/MonCat/Adjunctions.lean,Mathlib/Data/Finsupp/Option.lean,Mathlib/Data/Finsupp/Single.lean |
3 |
11 |
['BoltonBailey', 'eric-wieser', 'github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
4-6674 4 days ago |
4-6674 4 days ago |
6-30661 6 days |
25915 |
BoltonBailey author:BoltonBailey |
chore(Algebra/Squarefree/Basic): fix erw |
This PR addresses an instance of the erw linter in Algebra/Squarefree/Basic.
Original PR: https://github.com/leanprover-community/mathlib4/pull/25161 |
tech debt
t-algebra
easy
label:t-algebra$ |
1/1 |
Mathlib/Algebra/Squarefree/Basic.lean |
1 |
1 |
['github-actions'] |
nobody |
4-6491 4 days ago |
8-28413 8 days ago |
15-46477 15 days |
26195 |
yuanyi-350 author:yuanyi-350 |
add `Fin.cycleIcc` which rotates `range(i, j)` |
In this file, I define 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 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)
```
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-algebra
label:t-algebra$ |
161/1 |
Mathlib/Algebra/Group/Fin/Basic.lean,Mathlib/Data/Fin/Basic.lean,Mathlib/Data/Fin/SuccPred.lean,Mathlib/GroupTheory/Perm/Fin.lean |
4 |
1 |
['github-actions'] |
nobody |
3-80795 3 days ago |
10-73096 10 days ago |
10-84869 10 days |
25979 |
joelriou author:joelriou |
feat(CategoryTheory): the derived adjunction between absolute derived functors |
An adjunction between functors induces an adjunction between the corresponding left/right derived functors, when these derived functors are *absolute*, i.e. they remain derived functors after the post-composition with any functor.
This theorem is the generalized version by Georges Maltsiniotis (*Le théorème de Quillen, d'adjonction des
foncteurs dérivés, revisité*, C. R. Math. Acad. Sci. Paris 344 (2007), no. 9) of a theorem by Quillen for adjunctions between model categories.
---
This PR continues the work from #24144.
Original PR: https://github.com/leanprover-community/mathlib4/pull/24144 |
t-category-theory |
163/0 |
Mathlib.lean,Mathlib/CategoryTheory/Functor/Derived/Adjunction.lean,docs/references.bib |
3 |
3 |
['callesonne', 'github-actions', 'joelriou'] |
callesonne assignee:callesonne |
3-77230 3 days ago |
14-27634 14 days ago |
14-27679 14 days |
26036 |
joelriou author:joelriou |
feat(CategoryTheory/Functor): pointwise right derived functors |
This PR introduces pointwise right derived functors as particular cases of pointwise left Kan extensions.
---
This PR continues the work from #22490.
Original PR: https://github.com/leanprover-community/mathlib4/pull/22490 |
t-category-theory |
160/0 |
Mathlib.lean,Mathlib/CategoryTheory/Functor/Derived/PointwiseRightDerived.lean |
2 |
2 |
['github-actions', 'joelriou'] |
nobody |
3-77180 3 days ago |
13-50584 13 days ago |
13-50631 13 days |
26004 |
vasnesterov author:vasnesterov |
feat(Algebra/Order/Floor): `⌊n * x⌋₊ / n = ⌊x⌋₊` |
Prove that `⌊n * x⌋₊ / n = ⌊x⌋₊` for natural `n`.
---
[](https://gitpod.io/from-referrer/)
|
maintainer-merge
t-order
t-algebra
label:t-algebra$ |
39/9 |
Archive/Wiedijk100Theorems/SumOfPrimeReciprocalsDiverges.lean,Mathlib/Algebra/Order/Floor/Ring.lean,Mathlib/Algebra/Order/Floor/Semiring.lean,Mathlib/Data/EReal/Inv.lean |
4 |
21 |
['Ruben-VandeVelde', 'YaelDillies', 'b-mehta', 'eric-wieser', 'github-actions', 'vasnesterov'] |
nobody |
3-76923 3 days ago |
unknown |
unknown |
26302 |
kebekus author:kebekus |
feat: introduce the Laplace operator |
This PR continues the work from #25441.
Original PR: https://github.com/leanprover-community/mathlib4/pull/25441 |
t-analysis |
333/0 |
Mathlib.lean,Mathlib/Analysis/Calculus/ContDiff/Basic.lean,Mathlib/Analysis/Calculus/ContDiff/FTaylorSeries.lean,Mathlib/Analysis/InnerProductSpace/Laplace.lean |
4 |
37 |
['github-actions', 'grunweg', 'kebekus', 'sgouezel'] |
nobody |
3-75472 3 days ago |
3-75472 3 days ago |
5-49711 5 days |
24139 |
yuanyi-350 author:yuanyi-350 |
feat: add `Fin.cycleIcc` which rotates `range(i, j)` |
In this file, I define 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 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)
```
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-algebra
label:t-algebra$ |
132/1 |
Mathlib/Algebra/Group/Fin/Basic.lean,Mathlib/Data/Fin/Basic.lean,Mathlib/Data/Nat/SuccPred.lean,Mathlib/GroupTheory/Perm/Fin.lean |
4 |
44 |
['acmepjz', 'faenuccio', 'github-actions', 'grunweg', 'leanprover-bot', 'leanprover-community-bot-assistant', 'mbkybky', 'yuanyi-350'] |
faenuccio assignee:faenuccio |
3-74673 3 days ago |
3-74673 3 days ago |
73-78077 73 days |
26353 |
kebekus author:kebekus |
feat: restriction of scalars for iterated Fréchet derivatives |
Establish standard theorems on restriction of scalars for iterated Fréchet derivatives, comparing iterated derivatives with respect to a field `𝕜'` to iterated derivatives with respect to a subfield `𝕜 ⊆ 𝕜'`. The results are analogous to those found in
`Mathlib.Analysis.Calculus.FDeriv.RestrictScalars`.
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.
---
[](https://gitpod.io/from-referrer/)
|
t-analysis |
102/0 |
Mathlib.lean,Mathlib/Analysis/Calculus/ContDiff/Defs.lean,Mathlib/Analysis/Calculus/ContDiff/RestrictScalars.lean,Mathlib/Analysis/Calculus/FDeriv/RestrictScalars.lean |
4 |
4 |
['github-actions', 'kebekus', 'sgouezel'] |
nobody |
3-72997 3 days ago |
3-73088 3 days ago |
3-76644 3 days |
26426 |
Komyyy author:Komyyy |
doc: remove `PartENat.card` in the module doc |
[`PartENat.card`](https://leanprover-community.github.io/mathlib4_docs/Mathlib/Deprecated/Cardinal/Finite.html#PartENat.card) is moved to the `Deprecated` directory and it's not in this file([`Mathlib.SetTheory.Cardinal.Finite`](https://leanprover-community.github.io/mathlib4_docs/Mathlib/SetTheory/Cardinal/Finite.html)) anymore.
---
[](https://gitpod.io/from-referrer/)
|
t-set-theory
maintainer-merge
easy
documentation
|
0/2 |
Mathlib/SetTheory/Cardinal/Finite.lean |
1 |
2 |
['github-actions', 'grunweg'] |
nobody |
3-68563 3 days ago |
3-68563 3 days ago |
3-68577 3 days |
26396 |
xroblot author:xroblot |
feat(RingTheory): define the dual of a basis for the trace and prove basic properties |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
133/28 |
Mathlib/LinearAlgebra/BilinearForm/Properties.lean,Mathlib/RingTheory/DedekindDomain/Different.lean,Mathlib/RingTheory/Trace/Basic.lean |
3 |
1 |
['github-actions'] |
nobody |
3-58507 3 days ago |
5-73212 5 days ago |
5-73264 5 days |
26400 |
madvorak author:madvorak |
feat(Mathlib/Data/Fin/Pigeonhole): pigeonhole-like results for Fin |
Consider the following settings:
```
import Mathlib
example (X Y : Type) [Fintype X] [Fintype Y] (f : X → Y) (hf : f.Injective) :
Fintype.card X ≤ Fintype.card Y := by
hint
example (m n : ℕ) (f : Fin m → Fin n) (hf : f.Injective) :
m ≤ n := by
hint
example (X Y : Type) [Fintype X] [Fintype Y] (f : X ↪ Y) :
Fintype.card X ≤ Fintype.card Y := by
hint
example (m n : ℕ) (f : Fin m ↪ Fin n) :
m ≤ n := by
hint
```
The 1st and 3rd `hint` succeed, but the 2nd a 4th `hint` fail.
The problem is obviously that `exact?` does not see through `Fintype.card (Fin n) = n` when searching for appropriate lemma.
It may seem to not be a problem, as it will rarely derail experienced Mathlib users — after all, experienced Leaners usually go directly for the `Finset` or `Fintype` version.
However, beginners frequently work with `Fin` and they will expect stuff like
```
theorem le_of_injective (f : Fin m → Fin n) (hf : f.Injective) : m ≤ n
```
to exist; therefore, when `hint` or `exact?` fails, it is a very unpleasant surprise.
This PR addressed this issue; not to provide useful content for advanced users, but to make Mathlib more useful for beginners.
---
copied from #22792 where I lost push rights and needed to deprecate a name
[](https://gitpod.io/from-referrer/)
|
t-data |
58/0 |
Mathlib.lean,Mathlib/Data/Fin/Pigeonhole.lean |
2 |
9 |
['BoltonBailey', 'b-mehta', 'github-actions', 'madvorak'] |
nobody |
3-58485 3 days ago |
5-64037 5 days ago |
5-64092 5 days |
26474 |
xroblot author:xroblot |
feat(NumberTheory): `N(I 𝓞L) = N(I) ^ [L:K]` for an integral ideal `I` of `K` |
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-number-theory
|
74/4 |
Mathlib/NumberTheory/RamificationInertia/Basic.lean,Mathlib/RingTheory/DedekindDomain/Ideal.lean,Mathlib/RingTheory/Ideal/Int.lean,Mathlib/RingTheory/Ideal/Over.lean |
4 |
1 |
['github-actions'] |
nobody |
3-54803 3 days ago |
3-54811 3 days ago |
3-54863 3 days |
26453 |
jburroni author:jburroni |
feat(Data/PNat/Basic): add order-related instances to PNat |
Add `SuccAddOrder ℕ+` and `NoMaxOrder ℕ+` instances.
This allows, for example, the use of lemmas related to `Intervals` built with ℕ+.
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-data
new-contributor
|
18/0 |
Mathlib/Data/PNat/Basic.lean |
1 |
3 |
['eric-wieser', 'github-actions', 'jburroni'] |
nobody |
3-51546 3 days ago |
4-35404 4 days ago |
4-35451 4 days |
24778 |
YaelDillies author:YaelDillies |
feat: `CommGrp`-valued Yoneda embedding |
From Toric
Co-authored-by: Andrew Yang
---
[](https://gitpod.io/from-referrer/)
|
toric
t-category-theory
|
105/0 |
Mathlib.lean,Mathlib/Algebra/Category/Grp/Yoneda.lean,Mathlib/Algebra/Category/MonCat/Yoneda.lean,Mathlib/CategoryTheory/Preadditive/Yoneda/Basic.lean |
4 |
32 |
['TwoFX', 'YaelDillies', 'callesonne', 'erdOne', 'github-actions', 'kckennylau', 'leanprover-community-bot-assistant'] |
nobody |
3-39851 3 days ago |
20-42855 20 days ago |
47-53611 47 days |
26358 |
plp127 author:plp127 |
feat(Topology): R1 spaces are quasisober |
This PR continues the work from #24054.
Original PR: https://github.com/leanprover-community/mathlib4/pull/24054 |
bench-after-CI
t-topology
|
23/9 |
Mathlib/Topology/Separation/Hausdorff.lean,Mathlib/Topology/Sober.lean |
2 |
16 |
['faenuccio', 'github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'plp127'] |
nobody |
3-27260 3 days ago |
3-27316 3 days ago |
6-52291 6 days |
26280 |
AntoineChambert-Loir author:AntoineChambert-Loir |
feat(GroupTheory/GroupAction/Jordan) : Primitivity lemmas |
This is a primitivity lemma for actions, in preparation to the proof of of Jordan on primitive subgroups of the permutation group #26282
This PR continues the work from #24120.
Original PR: https://github.com/leanprover-community/mathlib4/pull/24120
- [ ] depends on: #26279
|
t-algebra label:t-algebra$ |
145/23 |
Mathlib/GroupTheory/GroupAction/MultiplePrimitivity.lean,Mathlib/GroupTheory/GroupAction/MultipleTransitivity.lean,Mathlib/GroupTheory/GroupAction/SubMulAction/OfFixingSubgroup.lean |
3 |
4 |
['AntoineChambert-Loir', 'github-actions', 'mathlib4-dependent-issues-bot', 'tb65536'] |
riccardobrasca assignee:riccardobrasca |
3-26309 3 days ago |
4-1802 4 days ago |
7-962 7 days |
26023 |
Garmelon author:Garmelon |
chore: add githelper.py script |
As described in the readme file, this somewhat opinionated script aims to help fix weird git repo setups and restore them to a standardized state that closely matches what `gh repo clone` does. Like `migrate_to_fork.py`, this script requires the user to have `git` and `gh` installed.
To use the script, run `scripts/githelper.py fix` in a git repo that is either a clone of mathlib or of a mathlib fork. The script will prompt you before making any changes, so the user retains control over the entire process. The script also prints the commands used.
`fix` is a subcommand so other git and github management tasks can be added in the future. Possible examples: Deleting branches of closed PRs, keeping the fork in sync with upstream, removing branches from a fork that was accidentally cloned with all mathlib branches included.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor |
490/0 |
scripts/README.md,scripts/githelper.py |
2 |
8 |
['Garmelon', 'bryangingechen', 'github-actions', 'jcommelin'] |
bryangingechen assignee:bryangingechen |
3-12189 3 days ago |
3-12189 3 days ago |
5-21466 5 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 |
3-11400 3 days ago |
6-33478 6 days ago |
6-33527 6 days |
26486 |
DavidLedvinka author:DavidLedvinka |
feat(Order): Add curried versions of `biSup_prod` and `biInf_prod` |
Used in the Brownian Motion project. |
t-order
easy
|
8/0 |
Mathlib/Order/CompleteLattice/Basic.lean |
1 |
1 |
['github-actions'] |
nobody |
3-863 3 days ago |
3-897 3 days ago |
3-910 3 days |
26469 |
euprunin author:euprunin |
chore: golf using `assumption_mod_cast` |
|
|
5/9 |
Mathlib/Algebra/Lie/Weights/Killing.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Arctan.lean,Mathlib/RingTheory/Norm/Defs.lean,Mathlib/Topology/Category/LightProfinite/Sequence.lean |
4 |
4 |
['bryangingechen', 'github-actions', 'leanprover-bot'] |
nobody |
2-79125 2 days ago |
2-79125 2 days ago |
3-62683 3 days |
26150 |
YaelDillies author:YaelDillies |
feat: `CanLift` instance from `ConvexCone` to `ProperCone` |
For this, move `ConvexCone.pointed_of_nonempty_of_mem` earlier and rename it to `ConvexCone.Pointed.of_nonempty_of_mem`.
From Toric
---
[](https://gitpod.io/from-referrer/)
|
toric
t-analysis
|
45/22 |
Mathlib/Analysis/Convex/Cone/Basic.lean,Mathlib/Analysis/Convex/Cone/InnerDual.lean |
2 |
4 |
['YaelDillies', 'b-mehta', 'github-actions'] |
nobody |
2-78519 2 days ago |
11-58148 11 days ago |
11-58441 11 days |
26033 |
joelriou author:joelriou |
feat(CategoryTheory/Abelian): isomorphisms modulo a Serre class |
---
This PR continues the work from #22739.
Original PR: https://github.com/leanprover-community/mathlib4/pull/22739 |
t-category-theory |
192/0 |
Mathlib.lean,Mathlib/CategoryTheory/Abelian/SerreClass/MorphismProperty.lean,Mathlib/CategoryTheory/Limits/Shapes/Equalizers.lean,Mathlib/CategoryTheory/Limits/Shapes/Kernels.lean,Mathlib/CategoryTheory/Preadditive/Basic.lean |
5 |
2 |
['github-actions', 'joelriou'] |
robin-carlier assignee:robin-carlier |
2-74732 2 days ago |
13-51810 13 days ago |
13-51856 13 days |
26272 |
ajirving author:ajirving |
feat(NumberTheory/LucasLehmer): prove converse direction to Lucas-Lehmer |
Proves the converse direction of the Lucas-Lehmer test, namely that the Lucas-Lehmer criterion is a necessary condition for a Mersenne prime.
Adds a couple of examples of proving Mersenne numbers are composite using this.
Proves that if `2^p-1` is prime then `p` is prime.
---
* I wasn't sure how many examples to add given that there are many more Mersenne composites than primes.
* There are a number of annoying coercions between different rings, any simplifications will be appreciated.
[](https://gitpod.io/from-referrer/)
|
large-import
new-contributor
t-number-theory
|
226/5 |
Archive/Examples/MersennePrimes.lean,Mathlib/NumberTheory/LucasLehmer.lean |
2 |
12 |
['github-actions', 'kckennylau'] |
nobody |
2-64743 2 days ago |
8-46839 8 days ago |
8-46886 8 days |
26287 |
mbkybky author:mbkybky |
feat(Data/ENat/Lattice): coercion to `WithBot ℕ∞` commutes with `biSup` |
The coercion from `ℕ∞` to `WithBot ℕ∞` commutes with `biSup` and `biInf`.
---
[](https://gitpod.io/from-referrer/)
|
t-data |
19/0 |
Mathlib/Data/ENat/Lattice.lean |
1 |
1 |
['github-actions'] |
nobody |
2-42017 2 days ago |
7-85957 7 days ago |
8-7308 8 days |
26492 |
Komyyy author:Komyyy |
feat: Alexandrov discrete implies locally path-connected |
The primary motivation for this theorem is to deduce path-connectedness from connectedness in finite topological spaces:
```lean
import Mathlib.Topology.Connected.LocPathConnected
example {X : Type*} [TopologicalSpace X] [Finite X] [ConnectedSpace X] : PathConnectedSpace X := by
rw [pathConnectedSpace_iff_connectedSpace]; assumption
```
---
[](https://gitpod.io/from-referrer/)
|
t-topology |
22/0 |
Mathlib/Topology/AlexandrovDiscrete.lean,Mathlib/Topology/Connected/LocPathConnected.lean |
2 |
1 |
['github-actions'] |
nobody |
2-37323 2 days ago |
2-37323 2 days ago |
2-37444 2 days |
26462 |
PSchwahn author:PSchwahn |
feat(LinearAlgebra/Projection): add results about inverse of `Submodule.prodEquivOfIsCompl` |
Add two theorems `Submodule.prodEquivOfIsCompl_symm_apply` and `Submodule.prodEquivOfIsCompl_symm_add`, which are API for `Submodule.prodEquivOfIsCompl`.
We believe these theorems are useful; for example, we have used their statements in a [classification formalization project](https://github.com/LieLean/LowDimSolvClassification).
I am not sure whether the `prodEquivOfIsCompl_symm_apply` theorem should be tagged with `@[simp]`; this might lead to confluence issues. Opinions are welcome!
Co-authored by:
- [Viviana del Barco](https://github.com/vdelbarc)
- [Gustavo Infanti](https://github.com/GuQOliveira)
- [Exequiel Rivas](https://github.com/erivas)
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-algebra
label:t-algebra$ |
9/0 |
Mathlib/LinearAlgebra/Projection.lean |
1 |
5 |
['PSchwahn', 'github-actions', 'kckennylau'] |
nobody |
2-18756 2 days ago |
4-4390 4 days ago |
4-4517 4 days |
25862 |
zcyemi author:zcyemi |
feat(Geometry/Euclidean/Triangle): add law of sines |
---
Implement the vector and angle-at-point forms of the law of sines.
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #25174.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/25174* |
migrated-from-branch
new-contributor
t-euclidean-geometry
|
53/1 |
Mathlib/Geometry/Euclidean/Triangle.lean |
1 |
8 |
['eric-wieser', 'github-actions', 'jsm28', 'zcyemi'] |
nobody |
2-12585 2 days ago |
16-49056 16 days ago |
16-52998 16 days |
26489 |
chrisflav author:chrisflav |
refactor(RingTheory/RingHom): factor out proofs for `Algebra.FinitePresentation` |
The current way to use locality of a given property of algebras is to convert everything into the language of `RingHom`s and then for example the `RingHom.OfLocalizationSpanTarget` API. This has two disadvantages:
1. The ring hom property API fixes the universes of source and target to be the same, hence we unnecessarily lose out on some universe generality.
2. The results for `RingHom`s are proven by translating everything in terms of `Algebra`, so we duplicate the translation steps.
This PR refactors `RingHom.FinitePresentation` to do all locality proofs in the language of `Algebra`s and translate it into the corresponding `RingHom.OfLocalizationSpan{Target}` in the last step. We also streamline some of the translation proofs by unifying the API.
---
- [x] depends on: #22931
[](https://gitpod.io/from-referrer/)
This PR continues the work from #22930.
Original PR: https://github.com/leanprover-community/mathlib4/pull/22930 |
t-algebra label:t-algebra$ |
62/77 |
Mathlib/RingTheory/RingHom/FinitePresentation.lean |
1 |
4 |
['chrisflav', 'erdOne', 'github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
1-84065 1 day ago |
2-53218 2 days ago |
2-53267 2 days |
26506 |
sgouezel author:sgouezel |
feat: smooth Riemannian bundles |
Given a vector bundle over a manifold whose fibers are all endowed with a scalar product, we
say that this bundle is Riemannian if the scalar product depends smoothly on the base point.
We introduce a typeclass `[IsContMDiffRiemannianBundle IB n F E]` registering this property.
Under this assumption, we show that the scalar product of two smooth maps into the same fibers of
the bundle is a smooth function.
If the fibers of a bundle `E` have a preexisting topology (like the tangent bundle), one can not
assume additionally `[∀ b, InnerProductSpace ℝ (E b)]` as this would create diamonds. Instead,
use `[RiemannianBundle E]`, which endows the fibers with a scalar product while ensuring that
there is no diamond. We provide a constructor for `[RiemannianBundle E]` from a smooth family
of metrics, which registers automatically `[IsContMDiffRiemannianBundle IB n F E]`
---
[](https://gitpod.io/from-referrer/)
|
t-differential-geometry |
201/0 |
Mathlib.lean,Mathlib/Geometry/Manifold/VectorBundle/Riemannian.lean |
2 |
1 |
['github-actions'] |
nobody |
1-81683 1 day ago |
1-81746 1 day ago |
1-81732 1 day |
22662 |
plp127 author:plp127 |
feat: Localization.Away.lift (computably) |
This PR adds `Localization.Away.lift'` and `Localization.Away.lift`, computable alternatives to `Localization.awayLift`.
---
- [x] depends on: #24791
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
74/0 |
Mathlib/RingTheory/Localization/Away/Basic.lean |
1 |
12 |
['eric-wieser', 'github-actions', 'mathlib4-dependent-issues-bot', 'plp127', 'vihdzp'] |
nobody |
1-81156 1 day ago |
50-16839 1 month ago |
116-16823 116 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 |
38/33 |
Mathlib/Tactic/Widget/LibraryRewrite.lean,MathlibTest/LibraryRewrite.lean |
2 |
3 |
['YaelDillies', 'erdOne', 'github-actions'] |
nobody |
1-76542 1 day ago |
3-48289 3 days ago |
3-48333 3 days |
26500 |
sgouezel author:sgouezel |
feat: more properties of the manifold structure on `Icc` |
The manifold structure on real intervals is defined in `Mathlib.Geometry.Manifold.Instances.Real`.
We relate it to the manifold structure on the real line, by showing that the inclusion and
projection are smooth, and showing that a function defined on the interval is smooth iff
its composition with the projection is smooth on the interval in `ℝ`.
We also define `1 : TangentSpace (𝓡∂ 1) z`, and relate it to `1` in the real line.
---
[](https://gitpod.io/from-referrer/)
|
t-differential-geometry |
215/2 |
Mathlib.lean,Mathlib/Geometry/Manifold/Instances/Icc.lean,Mathlib/Topology/Order/ProjIcc.lean |
3 |
9 |
['github-actions', 'grunweg', 'sgouezel'] |
grunweg assignee:grunweg |
1-75091 1 day ago |
1-75152 1 day ago |
1-82473 1 day |
26251 |
YaelDillies author:YaelDillies |
chore(Units): better follow the naming convention |
Moves
* `Units.ext` -> `Units.val_injective`
* `Units.eq_iff` -> `Units.val_inj`
---
[](https://gitpod.io/from-referrer/)
|
|
63/57 |
Mathlib/Algebra/GCDMonoid/Basic.lean,Mathlib/Algebra/Group/Center.lean,Mathlib/Algebra/Group/Units/Defs.lean,Mathlib/Algebra/Order/Monoid/Units.lean,Mathlib/Algebra/Polynomial/UnitTrinomial.lean,Mathlib/Algebra/Ring/Units.lean,Mathlib/Analysis/Complex/Isometry.lean,Mathlib/Data/Complex/Determinant.lean,Mathlib/Data/Fintype/Units.lean,Mathlib/Data/ZMod/Units.lean,Mathlib/FieldTheory/Finite/Basic.lean,Mathlib/GroupTheory/OrderOfElement.lean,Mathlib/LinearAlgebra/CliffordAlgebra/SpinGroup.lean,Mathlib/LinearAlgebra/Determinant.lean,Mathlib/LinearAlgebra/Lagrange.lean,Mathlib/LinearAlgebra/Matrix/SpecialLinearGroup.lean,Mathlib/NumberTheory/ArithmeticFunction.lean,Mathlib/NumberTheory/DirichletCharacter/Basic.lean,Mathlib/NumberTheory/DirichletCharacter/GaussSum.lean,Mathlib/NumberTheory/LucasPrimality.lean,Mathlib/NumberTheory/MulChar/Basic.lean,Mathlib/NumberTheory/NumberField/Units/Basic.lean,Mathlib/RingTheory/ClassGroup.lean,Mathlib/RingTheory/Fintype.lean,Mathlib/RingTheory/IntegralDomain.lean,Mathlib/RingTheory/RootsOfUnity/Basic.lean,Mathlib/RingTheory/RootsOfUnity/EnoughRootsOfUnity.lean,Mathlib/RingTheory/Valuation/RankOne.lean,Mathlib/Topology/Algebra/Constructions.lean,Mathlib/Topology/Algebra/IsOpenUnits.lean,MathlibTest/instance_diamonds.lean |
31 |
1 |
['github-actions'] |
nobody |
1-73061 1 day ago |
1-73078 1 day ago |
9-55700 9 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$ |
108/99 |
Mathlib/Data/Matrix/Basis.lean,Mathlib/RingTheory/MatrixAlgebra.lean |
2 |
12 |
['Whysoserioushah', 'eric-wieser', 'github-actions'] |
nobody |
1-61366 1 day ago |
3-11505 3 days ago |
19-67310 19 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$ |
275/4 |
Mathlib.lean,Mathlib/Analysis/NormedSpace/PiTensorProduct/ProjectiveSeminorm.lean,Mathlib/Data/Set/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 |
8 |
['eric-wieser', 'github-actions', 'joelriou'] |
nobody |
1-60228 1 day ago |
1-60228 1 day ago |
2-36990 2 days |
26502 |
sgouezel author:sgouezel |
feat: monotonicity of `lineMap` |
Also remove one assumption in `differentiableOn_integral_of_continuous`, and expand docstrings around this theorem.
---
[](https://gitpod.io/from-referrer/)
|
maintainer-merge
t-analysis
|
49/10 |
Mathlib/LinearAlgebra/AffineSpace/AffineMap.lean,Mathlib/MeasureTheory/Integral/IntervalIntegral/FundThmCalculus.lean,Mathlib/MeasureTheory/Integral/IntervalIntegral/IntegrationByParts.lean,Mathlib/Topology/Algebra/ContinuousAffineMap.lean |
4 |
6 |
['eric-wieser', 'github-actions', 'grunweg', 'sgouezel'] |
nobody |
1-58382 1 day ago |
1-77573 1 day ago |
1-83173 1 day |
26501 |
sgouezel author:sgouezel |
feat: more API on manifolds |
---
[](https://gitpod.io/from-referrer/)
|
t-differential-geometry |
65/7 |
Mathlib/Geometry/Manifold/IsManifold/Basic.lean,Mathlib/Geometry/Manifold/IsManifold/ExtChartAt.lean,Mathlib/Geometry/Manifold/MFDeriv/Atlas.lean,Mathlib/Geometry/Manifold/VectorBundle/Tangent.lean |
4 |
9 |
['github-actions', 'grunweg', 'sgouezel'] |
grunweg assignee:grunweg |
1-58036 1 day ago |
1-83577 1 day ago |
1-83563 1 day |
25781 |
emilyriehl author:emilyriehl |
Feat(CategoryTheory): terminal categories with an application to hoFunctor |
Some preliminary API around terminal categories is developed with an application for the infinity-cosmos project: proving that the homotopy category functor preserves terminal objects. We also include proofs that `[0]` is terminal in the simplex category and `Δ[0]` is the terminal simplicial set.
Co-authored by [Robin Carlier](robin.carlier@ens-lyon.fr), [Jakob von Raumer](https://github.com/javra), [Adam Topaz](topaz@ualberta.ca), and [Zeyi Zhao](zzhao95@jh.edu).
---
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #25459.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/25459* |
infinity-cosmos
large-import
t-category-theory
|
168/2 |
Mathlib.lean,Mathlib/AlgebraicTopology/SimplexCategory/Basic.lean,Mathlib/AlgebraicTopology/SimplicialSet/HomotopyCat.lean,Mathlib/AlgebraicTopology/SimplicialSet/Monoidal.lean,Mathlib/CategoryTheory/Category/Cat/Terminal.lean,Mathlib/CategoryTheory/Category/ReflQuiv.lean,Mathlib/CategoryTheory/Quotient.lean |
7 |
16 |
['emilyriehl', 'github-actions', 'joelriou'] |
nobody |
1-56620 1 day ago |
1-56620 1 day ago |
3-8949 3 days |
25970 |
wwylele author:wwylele |
feat(RingTheory): decompose archimedean classes of HahnSeries |
In preparation for #25140, this connects archimedean class and HahnSeries
---
[](https://gitpod.io/from-referrer/)
|
large-import |
494/2 |
Mathlib.lean,Mathlib/Algebra/Order/Archimedean/Class.lean,Mathlib/Order/Hom/Basic.lean,Mathlib/Order/Hom/Lex.lean,Mathlib/Order/Hom/WithTopBot.lean,Mathlib/RingTheory/HahnSeries/Lex.lean |
6 |
2 |
['ScottCarnahan', 'github-actions'] |
nobody |
1-52606 1 day ago |
14-35474 14 days ago |
14-35519 14 days |
25782 |
emilyriehl author:emilyriehl |
feat(CategoryTheory/Category/Cat): cartesian closed instance on small categories |
The category of small categories is cartesian closed, with exponentials defined by functor categories. Adjoint transposition is defined by currying and uncurrying.
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #25646.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/25646* |
infinity-cosmos
t-category-theory
|
160/1 |
Mathlib.lean,Mathlib/CategoryTheory/Category/Cat.lean,Mathlib/CategoryTheory/Category/Cat/CartesianClosed.lean,Mathlib/CategoryTheory/Functor/Currying.lean |
4 |
11 |
['callesonne', 'emilyriehl', 'github-actions', 'joelriou'] |
nobody |
1-51530 1 day ago |
1-51742 1 day ago |
3-73926 3 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 |
1-50822 1 day ago |
1-50848 1 day ago |
1-50895 1 day |
25784 |
emilyriehl author:emilyriehl |
feat(Bicategory/CatEnriched): 2-cat from Cat-enriched cat |
A construction of the canonical strict bicategory structure given a `EnrichedCategory Cat C`.
From the ∞-cosmos project.
Co-Authored-By: Emily Riehl
---
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #25287.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/25287* |
infinity-cosmos
t-category-theory
|
341/0 |
Mathlib.lean,Mathlib/CategoryTheory/Bicategory/CatEnriched.lean,Mathlib/CategoryTheory/Monoidal/Cartesian/Cat.lean |
3 |
4 |
['emilyriehl', 'github-actions', 'joelriou'] |
nobody |
1-50021 1 day ago |
1-50021 1 day ago |
2-10856 2 days |
26509 |
pechersky author:pechersky |
feat(RingTheory/Valuation): IsNontrivial.exists_one_lt |
And provide instance of IsNontrivial for RankOne.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-analysis
t-number-theory
label:t-algebra$ |
33/1 |
Mathlib/RingTheory/Valuation/Basic.lean,Mathlib/RingTheory/Valuation/RankOne.lean |
2 |
1 |
['github-actions'] |
nobody |
1-49452 1 day ago |
1-51382 1 day ago |
1-51399 1 day |
26511 |
pechersky author:pechersky |
feat(RingTheory/Valuation): le_one_of_subsingleton |
to provide `nontriviality` a helper simp lemma
---
[](https://gitpod.io/from-referrer/)
|
t-analysis
t-number-theory
easy
|
5/0 |
Mathlib/RingTheory/Valuation/Basic.lean |
1 |
1 |
['github-actions'] |
nobody |
1-49430 1 day ago |
1-49430 1 day ago |
1-49483 1 day |
26512 |
pechersky author:pechersky |
feat(RingTheory/Valuation/Integers): nontrivial_iff |
valuation subring is nontrivial iff ring is nontrivial
stated using Integers to be more general
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-analysis
t-number-theory
easy
label:t-algebra$ |
13/0 |
Mathlib/RingTheory/Valuation/Integers.lean |
1 |
1 |
['github-actions'] |
nobody |
1-49370 1 day ago |
1-49413 1 day ago |
1-49429 1 day |
26314 |
kckennylau author:kckennylau |
feat: Finsupp.supportedEquivFinsupp_symm_single |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
15/1 |
Mathlib/Data/Finsupp/Basic.lean,Mathlib/LinearAlgebra/Finsupp/Supported.lean |
2 |
8 |
['eric-wieser', 'github-actions', 'kckennylau'] |
nobody |
1-48262 1 day ago |
1-48663 1 day ago |
3-23208 3 days |
26060 |
kckennylau author:kckennylau |
feat(RingTheory): define Grassmannians |
This defines the Grassmannians of a module over a ring.
---
Zulip discussion: [#maths > Projective Space](https://leanprover.zulipchat.com/#narrow/channel/116395-maths/topic/Projective.20Space/with/524057860)
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-algebraic-geometry
label:t-algebra$ |
94/0 |
Mathlib.lean,Mathlib/RingTheory/Grassmannian.lean,docs/references.bib |
3 |
29 |
['erdOne', 'eric-wieser', 'github-actions', 'kckennylau', 'mattrobball'] |
nobody |
1-48181 1 day ago |
13-10473 13 days ago |
13-15035 13 days |
24350 |
erdOne author:erdOne |
feat(FieldTheory): fg extension over perfect field is separably generated |
Co-authored-by: Christian Merten
---
- [x] depends on: #24344
- [x] depends on: #24346
- [x] depends on: #24347
- [x] depends on: #24348
- [x] depends on: #24349
- [x] depends on: #25062
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
466/0 |
Mathlib.lean,Mathlib/FieldTheory/IntermediateField/Algebraic.lean,Mathlib/FieldTheory/SeparableClosure.lean,Mathlib/FieldTheory/SeparablyGenerated.lean,Mathlib/RingTheory/AlgebraicIndependent/Basic.lean,Mathlib/RingTheory/AlgebraicIndependent/TranscendenceBasis.lean |
6 |
29 |
['alreadydone', 'erdOne', 'github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
1-36976 1 day ago |
17-67971 17 days ago |
17-67969 17 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 |
4 |
['YaelDillies', 'eric-wieser', 'github-actions', 'robin-carlier'] |
nobody |
1-33255 1 day ago |
1-64705 1 day ago |
2-11375 2 days |
26114 |
wwylele author:wwylele |
feat(Data/Real): add embedding of archimedean groups into Real |
This is part of https://github.com/leanprover-community/mathlib4/pull/25140, and is the special case of Hahn embedding theorem applied to archimedean group.
----
This PR continues the work from #25157.
Original PR: https://github.com/leanprover-community/mathlib4/pull/25157 |
t-data |
231/0 |
Mathlib.lean,Mathlib/Data/Rat/Lemmas.lean,Mathlib/Data/Real/Embedding.lean |
3 |
21 |
['ScottCarnahan', 'github-actions', 'wwylele'] |
nobody |
1-32243 1 day ago |
12-38977 12 days ago |
12-39025 12 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 |
1-32103 1 day ago |
6-74841 6 days ago |
6-74884 6 days |
26347 |
mans0954 author:mans0954 |
feature(Data/Finset/RangeDistance): abs_sub_lt_of_mem_finset_range |
This PR continues the work from #23161.
Original PR: https://github.com/leanprover-community/mathlib4/pull/23161 |
|
30/0 |
Mathlib.lean,Mathlib/Algebra/Order/Group/Unbundled/Abs.lean,Mathlib/Data/Finset/RangeDistance.lean |
3 |
2 |
['github-actions', 'mans0954'] |
nobody |
1-31899 1 day ago |
6-75267 6 days ago |
6-75250 6 days |
26224 |
mans0954 author:mans0954 |
feature(Algebra/Polynomial/Roots) : nthRoots_two_one |
This PR continues the work from #24828.
Original PR: https://github.com/leanprover-community/mathlib4/pull/24828 |
|
5/0 |
Mathlib/Algebra/Polynomial/Roots.lean |
1 |
3 |
['github-actions', 'kckennylau', 'mans0954'] |
nobody |
1-30906 1 day ago |
10-48201 10 days ago |
10-48184 10 days |
25907 |
mans0954 author:mans0954 |
Low order roots of unity |
This PR continues the work from #25470.
Original PR: https://github.com/leanprover-community/mathlib4/pull/25470 |
t-algebra label:t-algebra$ |
182/0 |
Mathlib/Algebra/CharP/Invertible.lean,Mathlib/RingTheory/RootsOfUnity/Complex.lean |
2 |
2 |
['github-actions', 'mans0954'] |
nobody |
1-30833 1 day ago |
15-57908 15 days ago |
15-57959 15 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 |
1-30745 1 day ago |
15-58361 15 days ago |
15-58406 15 days |
26524 |
pechersky author:pechersky |
chore(RingTheory/Valuation): Valution.Integers implies IsFractionRing |
generalize `IsFractionRing v.integer K` to `IsFractionRing O K` when `v.Integers O K`.
Since `IsFractionRing` is prop, one should have a prop-relationship between the valuation subring and base ring
On the way, remove `IsDomain O` from the necessary TC arguments, since it is implied by `Valuation.Integers`
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
35/22 |
Mathlib/RingTheory/Valuation/ValuationRing.lean |
1 |
1 |
['github-actions'] |
nobody |
1-29054 1 day ago |
1-29065 1 day ago |
1-29107 1 day |
26006 |
CBirkbeck author:CBirkbeck |
Add the Mittag-Leffler expansion for cotangent |
This PR continues the work from #25448.
Original PR: https://github.com/leanprover-community/mathlib4/pull/25448 |
large-import |
187/3 |
Mathlib/Analysis/Complex/IntegerCompl.lean,Mathlib/Analysis/Complex/LocallyUniformLimit.lean,Mathlib/Analysis/SpecialFunctions/Log/Summable.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Cotangent.lean |
4 |
1 |
['github-actions'] |
nobody |
1-24073 1 day ago |
1-34475 1 day ago |
13-68841 13 days |
25348 |
wwylele author:wwylele |
feat(LinearAlgebra): add independent iSup to LinearPMap |
This is part of #25140. To obtain the Hahn embedding, we need to construct an partial linear map spanned by a family of submodules as the base case. This PR prepares for it.
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebra
label:t-algebra$ |
94/2 |
Mathlib/LinearAlgebra/DFinsupp.lean,Mathlib/LinearAlgebra/LinearPMap.lean |
2 |
3 |
['eric-wieser', 'github-actions', 'wwylele'] |
nobody |
1-13150 1 day ago |
29-39582 29 days ago |
29-39645 29 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 |
473/0 |
Mathlib.lean,Mathlib/Geometry/Diffeology/Basic.lean,docs/references.bib,scripts/noshake.json |
4 |
7 |
['JovanGerb', 'github-actions', 'lecopivo', 'peabrainiac'] |
nobody |
1-12847 1 day ago |
3-5302 3 days ago |
3-10056 3 days |
26488 |
yuanyi-350 author:yuanyi-350 |
add some lemmas about `Nat.gcd` |
add some lemmas about `Nat.gcd`
$lcm(\frac{k}{m}, \frac{k}{n}) = k / \gcd(m, n)$
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
easy
label:t-algebra$ |
24/1 |
Mathlib/Data/Nat/GCD/Basic.lean |
1 |
2 |
['github-actions', 'wwylele'] |
nobody |
1-10219 1 day ago |
2-62413 2 days ago |
2-62614 2 days |
26166 |
joelriou author:joelriou |
feat(AlgebraicTopology): application of the retract argument to model categories |
Basic consequences of the retract argument are obtained for model categories: cofibrations are exactly the morphisms that have the left lifting property with respect to trivial fibrations, etc. We deduce various properties of cofibrations, fibrations and weak equivalences in model categories (e.g. they are stable by composition).
---
(I am sorry if this one is a little bit long. There are too many basic properties to state.)
This PR continues the work from #20210.
Original PR: https://github.com/leanprover-community/mathlib4/pull/20210 |
large-import
maintainer-merge
t-topology
|
450/4 |
Mathlib.lean,Mathlib/AlgebraicTopology/ModelCategory/Basic.lean,Mathlib/AlgebraicTopology/ModelCategory/Instances.lean |
3 |
n/a |
['github-actions', 'joelriou', 'robin-carlier'] |
robin-carlier assignee:robin-carlier |
0-79620 22 hours ago |
unknown |
unknown |
26204 |
Raph-DG author:Raph-DG |
feat(AlgebraicGeometry): Add global preorder instance for schemes |
In this PR we added a default preorder instance for schemes, defined to be the specialization order as discussed here: https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/dimension.20function.20for.20schemes/near/524997376 for discussion
---
[](https://gitpod.io/from-referrer/)
|
t-algebraic-geometry
easy
|
15/0 |
Mathlib/AlgebraicGeometry/AffineSpace.lean,Mathlib/AlgebraicGeometry/Scheme.lean |
2 |
3 |
['Raph-DG', 'erdOne', 'github-actions'] |
nobody |
0-74359 20 hours ago |
6-58163 6 days ago |
9-76714 9 days |
24361 |
Hagb author:Hagb |
feat(Data/Finsupp/MonomialOrder): `0 ≤ a` where `a : m.syn` |
`simp` would be able to solve it.
---
[](https://gitpod.io/from-referrer/)
|
t-data
maintainer-merge
new-contributor
easy
|
3/0 |
Mathlib/Data/Finsupp/MonomialOrder.lean |
1 |
2 |
['Ruben-VandeVelde', 'github-actions'] |
nobody |
0-73516 20 hours ago |
0-73516 20 hours ago |
66-74278 66 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/)
|
t-algebra label:t-algebra$ |
11/0 |
Mathlib/RingTheory/Ideal/Operations.lean,Mathlib/RingTheory/Ideal/Span.lean |
2 |
1 |
['github-actions'] |
nobody |
0-73190 20 hours ago |
11-62777 11 days ago |
11-62808 11 days |
26531 |
JovanGerb author:JovanGerb |
fix(RefinedDiscrTree): remove funny `transparency` handling |
This PR fixes some funny behaviour of `RefinedDiscrTree` discovered at #26484.
This PR aligns the behaviour with Lean core's `DiscrTree`. The original reason for this special treatment was to avoid a mathlib breakage. But now it turns out that this special trearment also causes a mathlib breakage (but this one is harder to fix).
The breakage that was the original reason for this behaviour is easily fixed using a `dsimp`.
#26484 depends on this PR
---
[](https://gitpod.io/from-referrer/)
|
t-meta |
6/13 |
Mathlib/Lean/Meta/RefinedDiscrTree/Basic.lean,Mathlib/Lean/Meta/RefinedDiscrTree/Encode.lean,Mathlib/Probability/ProductMeasure.lean |
3 |
2 |
['github-actions', 'grunweg'] |
nobody |
0-71271 19 hours ago |
1-15026 1 day ago |
1-15072 1 day |
26536 |
peterjunglas author:peterjunglas |
fix (Data/Matrix/Rank): extend applicability of rank_submatrix_le |
The current version of `rank_submatrix_le` is restricted to square matrices and doesn't allow for the reduction of lines. Both restrictions can be removed easily without changing the proof.
---
[](https://gitpod.io/from-referrer/)
|
t-data
new-contributor
|
3/2 |
Mathlib/Data/Matrix/Rank.lean |
1 |
1 |
['github-actions'] |
nobody |
0-70435 19 hours ago |
0-70843 19 hours ago |
0-70888 19 hours |
24582 |
pechersky author:pechersky |
feat(GroupTheory/ArchimedeanDensely): Unique (ℤ ≃+o ℤ) |
---
[](https://gitpod.io/from-referrer/)
- [x] depends on: #24580 |
maintainer-merge
t-order
t-algebra
label:t-algebra$ |
44/0 |
Mathlib/Data/Int/Cast/Lemmas.lean,Mathlib/GroupTheory/ArchimedeanDensely.lean |
2 |
6 |
['Ruben-VandeVelde', 'eric-wieser', 'github-actions', 'mathlib4-dependent-issues-bot', 'pechersky'] |
nobody |
0-70407 19 hours ago |
0-70407 19 hours ago |
36-58613 36 days |
25758 |
YaelDillies author:YaelDillies |
chore: shortcut instance `CompleteLattice α → PartialOrder α` |
This avoids using the path `CompleteLattice α → CompletePartialOrder α → PartialOrder α` that goes through `Order.CompletePartialOrder` and makes it appear used to our automation, such as `shake` or `#min_imports`.
This is a followup to #25358.
---
[](https://gitpod.io/from-referrer/)
|
maintainer-merge
t-order
|
7/0 |
Mathlib/Order/CompleteLattice/Defs.lean |
1 |
2 |
['Ruben-VandeVelde', 'github-actions'] |
nobody |
0-70298 19 hours ago |
0-70298 19 hours ago |
18-70786 18 days |
25897 |
YaelDillies author:YaelDillies |
feat: `ofNat(n) • a = ofNat(n) * a` |
From Toric
---
[](https://gitpod.io/from-referrer/)
|
toric
t-data
maintainer-merge
t-algebra
label:t-algebra$ |
3/0 |
Mathlib/Data/Nat/Cast/Basic.lean |
1 |
2 |
['Ruben-VandeVelde', 'github-actions'] |
nobody |
0-70177 19 hours ago |
0-70177 19 hours ago |
15-67687 15 days |
24172 |
LessnessRandomness author:LessnessRandomness |
feat: specialize rational root theorem to usual rational numbers and integers |
Rational root theorem and integral root theorem - the special case for usual rational numbers and integers.
--- |
new-contributor
t-algebra
label:t-algebra$ |
123/0 |
Mathlib.lean,Mathlib/RingTheory/Polynomial/OfRationalNumbers/RationalRootTheorem.lean |
2 |
4 |
['Pazzaz', 'github-actions', 'grunweg', 'mariainesdff'] |
nobody |
0-70040 19 hours ago |
73-44288 2 months ago |
73-44341 73 days |
26297 |
mbkybky author:mbkybky |
feat(RingTheory): lemmas about `TensorProduct` and `IsBaseChange` |
Add lemmas about `TensorProduct` and `IsBaseChange`.
These are used to prove that [RingTheory.Sequence.IsWeaklyRegular](https://leanprover-community.github.io/mathlib4_docs/Mathlib/RingTheory/Regular/RegularSequence.html#RingTheory.Sequence.IsWeaklyRegular) is stable under flat base change and [RingTheory.Sequence.IsRegular](https://leanprover-community.github.io/mathlib4_docs/Mathlib/RingTheory/Regular/RegularSequence.html#RingTheory.Sequence.IsRegular) is stable under faithfully flat base change.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
65/10 |
Mathlib/LinearAlgebra/Quotient/Defs.lean,Mathlib/LinearAlgebra/TensorProduct/Basic.lean,Mathlib/LinearAlgebra/TensorProduct/Quotient.lean,Mathlib/RingTheory/Flat/FaithfullyFlat/Basic.lean,Mathlib/RingTheory/IsTensorProduct.lean,Mathlib/RingTheory/QuotSMulTop.lean |
6 |
1 |
['github-actions'] |
riccardobrasca assignee:riccardobrasca |
0-69672 19 hours ago |
7-59027 7 days ago |
7-62043 7 days |
26535 |
joelriou author:joelriou |
feat(Algebra/Homology/Embedding): the homology of the restriction |
Given an embedding of complex shapes, we provide an API to compute the homology of the "restriction".
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-category-theory
label:t-algebra$ |
122/0 |
Mathlib/Algebra/Homology/Embedding/RestrictionHomology.lean,Mathlib/Algebra/Homology/ShortComplex/HomologicalComplex.lean |
2 |
1 |
['github-actions'] |
nobody |
0-68019 18 hours ago |
0-71498 19 hours ago |
0-71541 19 hours |
26027 |
vasnesterov author:vasnesterov |
feat(Topology): every compact metric space can be embedded into the Hilbert cube |
Prove `exists_closed_embedding_to_hilbert_cube`: every compact metric space can be embedded into the Hilbert cube.
---
[](https://gitpod.io/from-referrer/)
|
maintainer-merge
t-topology
|
58/1 |
Mathlib.lean,Mathlib/Topology/Compactness/HilbertCubeEmbedding.lean,Mathlib/Topology/MetricSpace/Bounded.lean |
3 |
9 |
['ADedecker', 'github-actions', 'jcommelin', 'vasnesterov'] |
nobody |
0-67435 18 hours ago |
0-67435 18 hours ago |
13-49994 13 days |
26295 |
DavidJWebb author:DavidJWebb |
feat: filtering lists and bounded quantifiers are primitive recursive |
A few useful lemmas not explicitly in Primrec.lean :
- Filtering for elements from a list that meet a primrec criterion is primrec
- Checking whether a list has some element meeting a primrec criterion is primrec
- Checking whether every element of a list meets a primrec criterion is primrec
- Primitive recursive functions are closed under bounded existential and universal quantifiers
---
[](https://gitpod.io/from-referrer/)
|
t-computability
new-contributor
|
210/0 |
Mathlib.lean,Mathlib/Computability/PrimrecFilter.lean |
2 |
3 |
['DavidJWebb', 'github-actions', 'grunweg'] |
nobody |
0-67082 18 hours ago |
6-81644 6 days ago |
6-83335 6 days |
26537 |
mariainesdff author:mariainesdff |
feat(Analysis.Normed.Unbundled.SpectralNormUnique): prove unique extension theorem |
Let `K` be a field complete with respect to a nontrivial nonarchimedean multiplicative norm and `L/K` be an algebraic extension. We show that the spectral norm on `L` is a nonarchimedean multiplicative norm, and any power-multiplicative `K`-algebra norm on `L` coincides with the spectral norm. More over, if `L/K` is finite, then `L` is a complete space.
This result is [S. Bosch, U. Güntzer, R. Remmert,*Non-Archimedean Analysis* (Theorem 3.2.4/2)][bosch-guntzer-remmert].
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-analysis
|
247/0 |
Mathlib/Analysis/Normed/Unbundled/SpectralNorm.lean |
1 |
2 |
['github-actions', 'mariainesdff'] |
nobody |
0-66759 18 hours ago |
0-66767 18 hours ago |
0-66826 18 hours |
26373 |
b-mehta author:b-mehta |
chore(Finset/Card): cleanup section and improve documentation |
- Use the `Set.MapsTo` spelling (and similar) where possible, for consistency throughout mathlib
- Improve documentation on some lemmas ("reorder" has little meaning on finsets, which are inherently unordered)
- Add documentation to other lemmas
---
[](https://gitpod.io/from-referrer/)
|
t-data |
67/38 |
Mathlib/Combinatorics/Additive/Energy.lean,Mathlib/Combinatorics/Additive/PluenneckeRuzsa.lean,Mathlib/Combinatorics/Additive/VerySmallDoubling.lean,Mathlib/Combinatorics/SimpleGraph/Triangle/Counting.lean,Mathlib/Data/Finset/Card.lean,Mathlib/Data/Finset/Preimage.lean,Mathlib/Data/Setoid/Partition/Card.lean,Mathlib/NumberTheory/LegendreSymbol/GaussEisensteinLemmas.lean,Mathlib/NumberTheory/MaricaSchoenheim.lean,Mathlib/RingTheory/IntegralDomain.lean |
10 |
7 |
['b-mehta', 'github-actions', 'grunweg', 'jcommelin', 'mathlib-bors'] |
nobody |
0-65287 18 hours ago |
2-15653 2 days ago |
6-10266 6 days |
26365 |
joelriou author:joelriou |
feat(CategoryTheory/Localization): generalize results about adjunctions |
In this PR, results about adjunctions, localization of categories and calculus of fractions are slightly generalized. In particular, we show that under certain circumstances, adjoint functors are localization functors. (This shall be used in the proof of the fundamental lemma of homotopical algebra #26303.)
---
[](https://gitpod.io/from-referrer/)
|
t-category-theory |
108/25 |
Mathlib/CategoryTheory/Localization/CalculusOfFractions/OfAdjunction.lean,Mathlib/CategoryTheory/Localization/Opposite.lean |
2 |
3 |
['github-actions', 'joelriou', 'robin-carlier'] |
robin-carlier assignee:robin-carlier |
0-64645 17 hours ago |
6-45253 6 days ago |
6-45238 6 days |
26541 |
YaelDillies author:YaelDillies |
chore: rename `ZMod.natCast_zmod_eq_zero_iff_dvd` to `ZMod.natCast_eq_zero_iff` |
This matches `CharP.cast_eq_zero_iff`
---
[](https://gitpod.io/from-referrer/)
|
|
20/18 |
Archive/Imo/Imo2024Q2.lean,Archive/Wiedijk100Theorems/FriendshipGraphs.lean,Mathlib/Data/ZMod/Basic.lean,Mathlib/NumberTheory/Fermat.lean,Mathlib/NumberTheory/LucasLehmer.lean,Mathlib/NumberTheory/Padics/RingHoms.lean,Mathlib/NumberTheory/SumFourSquares.lean,Mathlib/NumberTheory/Wilson.lean,Mathlib/RingTheory/Fintype.lean,Mathlib/RingTheory/Polynomial/Cyclotomic/Basic.lean,Mathlib/RingTheory/RootsOfUnity/Minpoly.lean |
11 |
1 |
['github-actions'] |
nobody |
0-61782 17 hours ago |
0-61847 17 hours ago |
0-61831 17 hours |
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$ |
124/0 |
Mathlib.lean,Mathlib/LinearAlgebra/TensorPower/Symmetric.lean |
2 |
5 |
['AntoineChambert-Loir', 'erdOne', 'eric-wieser', 'github-actions'] |
nobody |
0-61446 17 hours ago |
11-16138 11 days ago |
11-16183 11 days |
26285 |
kckennylau author:kckennylau |
feat(RingTheory): resultant of two polynomials |
Co-authored-by: Anne Baanen
---
Split from #26283.
[](https://gitpod.io/from-referrer/)
|
maintainer-merge
t-algebra
label:t-algebra$ |
87/0 |
Mathlib.lean,Mathlib/RingTheory/Polynomial/Resultant/Basic.lean |
2 |
20 |
['MichaelStollBayreuth', 'YaelDillies', 'eric-wieser', 'github-actions', 'kckennylau'] |
nobody |
0-58942 16 hours ago |
0-60960 16 hours ago |
8-6725 8 days |
26504 |
sgouezel author:sgouezel |
feat: the image of an interval under a continuous monotone map is an interval |
---
[](https://gitpod.io/from-referrer/)
|
t-topology |
46/3 |
Mathlib/Order/ConditionallyCompleteLattice/Basic.lean,Mathlib/Topology/FiberBundle/Basic.lean,Mathlib/Topology/Order/Compact.lean |
3 |
6 |
['PatrickMassot', 'github-actions', 'sgouezel'] |
nobody |
0-58005 16 hours ago |
1-82363 1 day ago |
1-82348 1 day |
26411 |
sgouezel author:sgouezel |
feat: add `iInf` results on `ENNReal`, matching existing `iSup` ones |
---
[](https://gitpod.io/from-referrer/)
|
t-data |
39/0 |
Mathlib/Data/ENNReal/Operations.lean |
1 |
20 |
['YaelDillies', 'github-actions', 'grunweg', 'sgouezel'] |
nobody |
0-56146 15 hours ago |
0-56188 15 hours ago |
4-53043 4 days |
25743 |
robin-carlier author:robin-carlier |
feat(AlgebraicTopology/SimplexCategory/Augmented): monoidal structure on `AugmentedSimplexCategory` |
We construct a monoidal category structure on `AugmentedSimplexCategory`. The tensor products corresponds to ordinal sum. We characterize morphisms out of a tensor product of object in terms of their precomposition with canonical maps `x ⟶ x ⊗ y` and `y ⟶ x ⊗ y` coming from the fact that the unit is an initial object.
---
- [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.
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #22768.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/22768* |
t-topology
t-category-theory
|
512/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 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'robin-carlier'] |
nobody |
0-56004 15 hours ago |
15-38506 15 days ago |
15-38491 15 days |
26155 |
xroblot author:xroblot |
feat(DedekindDomain/Different): add the transitivity formula |
This PR proves the transitivity formula for the different ideal.
It introduces ~~two~~ one increase~~s~~ in imports:
- `RingTheory.FractionalIdeal.Extended`: this is a short leaf file and I think the import makes sense there
- ~~`RingTheory.Localization.Defs.lean `: the file `Algebra.Algebra.Basic` is added since it is necessary to have the definition of `noZeroSMulDivisors` to get that some algebra map is injective. The import could be removed by stating the hypothesis as `Function.Injective (algebraMap * *)` but it is not the usual spelling (and cannot be synthesized by Lean). In the end, it appears that the increased import only affects three files so maybe it's fine.~~
The PR also adds two new instances:
- `FiniteDimensional (FractionRing A) (FractionRing B)` deduced from `Module.Finite A B` when `B` is a Dedekind domain.
- `IsScalarTower (FractionRing A) (FractionRing B) (FractionRing C)` deduced from `IsScalarTower A B C`
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebra
label:t-algebra$ |
207/4 |
Mathlib/RingTheory/DedekindDomain/Different.lean,Mathlib/RingTheory/DedekindDomain/IntegralClosure.lean,Mathlib/RingTheory/FractionalIdeal/Extended.lean,Mathlib/RingTheory/Localization/Basic.lean,Mathlib/RingTheory/Localization/FractionRing.lean |
5 |
13 |
['erdOne', 'github-actions', 'xroblot'] |
nobody |
0-55454 15 hours ago |
3-56217 3 days ago |
8-53226 8 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 |
0-55150 15 hours ago |
9-74730 9 days ago |
17-19717 17 days |
26545 |
pechersky author:pechersky |
chore(RingTheory/Valuation): generalize lemmas about valuation of irreducibles in subring |
To prepare for generalization of LocallyCompact to Valued from NormedField
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-analysis
t-number-theory
label:t-algebra$ |
94/33 |
Mathlib/RingTheory/DiscreteValuationRing/Basic.lean,Mathlib/RingTheory/Valuation/Integers.lean,Mathlib/Topology/Algebra/Valued/LocallyCompact.lean |
3 |
1 |
['github-actions'] |
nobody |
0-51521 14 hours ago |
0-51569 14 hours ago |
0-51576 14 hours |
26546 |
101damnations author:101damnations |
refactor: denote low degree group cohomology API indices with subscripts |
This PR replaces names like `groupCohomology.oneCocycles` with `groupCohomology.cocycles₁`, to bring this API in line with the group homology naming scheme suggested by @jcommelin in #25873.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
594/352 |
Mathlib/RepresentationTheory/Homological/GroupCohomology/Functoriality.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/Hilbert90.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/LowDegree.lean |
3 |
1 |
['github-actions'] |
nobody |
0-51320 14 hours ago |
0-51325 14 hours ago |
0-51375 14 hours |
26522 |
Ruben-VandeVelde author:Ruben-VandeVelde |
chore: split out NatCast/IntCast Complex instances |
This makes it possible to simplify some proofs
---
[](https://gitpod.io/from-referrer/)
|
t-data |
36/35 |
Mathlib/Data/Complex/Basic.lean |
1 |
8 |
['Ruben-VandeVelde', 'eric-wieser', 'github-actions'] |
nobody |
0-51050 14 hours ago |
0-71874 19 hours ago |
1-37372 1 day |
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 |
0-50631 14 hours ago |
6-54015 6 days ago |
6-54067 6 days |
26351 |
RemyDegenne author:RemyDegenne |
feat: covering and packing numbers of sets in a metric space |
We define covering numbers of sets in a pseudo-metric space, which are minimal cardinalities of
`ε`-covers of sets. We also define the packing number, which is the maximal cardinality of
an `ε`-separated set.
From the Brownian motion project.
---
[](https://gitpod.io/from-referrer/)
|
t-topology |
261/0 |
Mathlib.lean,Mathlib/Topology/MetricSpace/CoveringNumbers.lean |
2 |
4 |
['ADedecker', 'YaelDillies', 'github-actions'] |
nobody |
0-50114 13 hours ago |
6-67740 6 days ago |
6-67787 6 days |
25882 |
101damnations author:101damnations |
feat(RepresentationTheory/Homological/GroupHomology/LowDegree): API for(one/two)(Cycles/Boundaries) |
This PR is more API for low degree group homology, adding (one/two)(Cycles/Boundaries), following the structure of `RepresentationTheory.Homological.GroupCohomology.LowDegree`.
---
- [x] depends on: #21652
- [x] depends on: #21732
- [x] depends on: #21733
- [x] depends on: #21735
- [x] depends on: #21736
- [x] depends on: #21738
- [ ] depends on: #25868
- [ ] depends on: #25873
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #21755.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/21755* |
file-removed
t-algebra
label:t-algebra$ |
691/19 |
Mathlib.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/Basic.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/Functoriality.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/Hilbert90.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/LowDegree.lean,Mathlib/RepresentationTheory/Homological/GroupHomology/Basic.lean,Mathlib/RepresentationTheory/Homological/GroupHomology/LowDegree.lean,Mathlib/RepresentationTheory/Homological/Resolution.lean |
8 |
n/a |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
0-49850 13 hours ago |
unknown |
unknown |
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/)
|
large-import
t-algebra
label:t-algebra$ |
356/2 |
Mathlib.lean,Mathlib/Data/Nat/Factorial/NatCast.lean,Mathlib/RingTheory/DividedPowers/RatAlgebra.lean |
3 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
0-49758 13 hours ago |
0-49760 13 hours ago |
3-32242 3 days |
26544 |
vihdzp author:vihdzp |
feat(SetTheory/ZFC/Ordinal): Lean ordinals to ZFC ordinals |
We define `Ordinal.toZFSet` and prove that its outputs are precisely the ZFC ordinals. Moved from #19985.
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-set-theory
|
151/4 |
Mathlib/SetTheory/ZFC/Basic.lean,Mathlib/SetTheory/ZFC/Ordinal.lean,Mathlib/SetTheory/ZFC/PSet.lean,Mathlib/SetTheory/ZFC/Rank.lean |
4 |
1 |
['github-actions'] |
nobody |
0-48805 13 hours ago |
0-51392 14 hours ago |
0-52775 14 hours |
26498 |
EtienneC30 author:EtienneC30 |
feat: projections and injections for WithLp |
Introduce `WithLp.fst` and `WithLp.snd` to avoid defeq abuse by writing `x.1` when `x : WithLp p (α × β)`. Also add a `ContinuousLinearMap` version.
Introduce `WithLp.inl` (resp. `WithLp.inr`) as a linear isometry from `α` (resp. β) to `WithLp p (α × β)`.
Introduce `PiLp.single` as a linear isometry from `β i` to `PiLp p β`.
---
[](https://gitpod.io/from-referrer/)
|
t-analysis |
107/7 |
Mathlib/Analysis/Normed/Lp/PiLp.lean,Mathlib/Analysis/Normed/Lp/ProdLp.lean,Mathlib/Analysis/Normed/Lp/WithLp.lean,Mathlib/LinearAlgebra/Pi.lean |
4 |
6 |
['EtienneC30', 'b-mehta', 'eric-wieser', 'github-actions'] |
nobody |
0-48385 13 hours ago |
1-50968 1 day ago |
2-16113 2 days |
26527 |
jsm28 author:jsm28 |
feat(LinearAlgebra/AffineSpace/Independent): `faceOpposite` point in 1-simplex |
Add a lemma about the point of `faceOpposite` applied to a 1-simplex.
```lean
lemma faceOpposite_point_eq_point_rev (s : Simplex k P 1) (i : Fin 2) (n : Fin 1) :
(s.faceOpposite i).points n = s.points i.rev := by
```
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
easy
label:t-algebra$ |
19/0 |
Mathlib/LinearAlgebra/AffineSpace/Independent.lean |
1 |
13 |
['eric-wieser', 'github-actions', 'jsm28'] |
nobody |
0-46437 12 hours ago |
1-22152 1 day ago |
1-22137 1 day |
26277 |
AntoineChambert-Loir author:AntoineChambert-Loir |
feat(RingTheory/Congruence/Hom): prove basic isomorphisms theorems for ring congruences |
This file contains elementary definitions involving congruence
relations and morphisms for semirings, rings, and algebras.
* `RingCon.ker`: the kernel of a monoid homomorphism as a congruence relation
* `RingCon.lift`, `RingCon.liftₐ`: the homomorphism / the algebra morphism
on the quotient given that the congruence is in the kernel
* `RingCon.map`, `RingCon.mapₐ`: homomorphism / algebra morphism
from a smaller to a larger quotient
* `RingCon.quotientKerEquivRangeS`, `RingCon.quotientKerEquivRange`,
`RingCon.quotientKerEquivRangeₐ` :
the first isomorphism theorem for semirings (using `RingHom.rangeS`),
rings (using `RingHom.range`) and algebras (using `AlgHom.range`).
* `RingCon.comapQuotientEquivRangeS`, `RingCon.comapQuotientEquivRange`,
`RingCon.comapQuotientEquivRangeₐ` : the second isomorphism theorem
for semirings (using `RingHom.rangeS`), rings (using `RingHom.range`)
and algebras (using `AlgHom.range`).
* `RingCon.quotientQuotientEquivQuotient`, `RingCon.quotientQuotientEquivQuotientₐ` :
the third isomorphism theorem for semirings (or rings) and algebras
It is an adaptation of what existed for multiplicative congruences (docs#Con) and is only useful for semirings which are not rings.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
555/2 |
Mathlib.lean,Mathlib/Algebra/Ring/Subsemiring/Basic.lean,Mathlib/Algebra/RingQuot.lean,Mathlib/RingTheory/Congruence/Basic.lean,Mathlib/RingTheory/Congruence/Defs.lean,Mathlib/RingTheory/Congruence/Hom.lean |
6 |
1 |
['github-actions'] |
nobody |
0-44989 12 hours ago |
8-24076 8 days ago |
8-24125 8 days |
26480 |
Citronhat author:Citronhat |
refactor(Data/NNRat/BigOperators): generalize `coe` big operator lemmas |
This refactor generalizes the `norm_cast` lemmas for sums and products of coercion of `ℚ≥0` elements.
Previously, these lemmas were stated only for coercion to `ℚ`. This change generalizes the target type `β` to any `[DivisionSemiring β]` with `[CharZero β]` for sums, and any `[Semifield β]` with `[CharZero β]` for products.
---
[](https://gitpod.io/from-referrer/)
|
t-data
new-contributor
|
44/16 |
Mathlib/Data/NNRat/BigOperators.lean |
1 |
10 |
['Citronhat', 'YaelDillies', 'eric-wieser', 'github-actions'] |
nobody |
0-44479 12 hours ago |
0-52012 14 hours ago |
2-40915 2 days |
25945 |
adomani author:adomani |
feat: the empty line in commands linter |
This linter flags empty lines within a command.
It allows empty lines within doc-strings, module-docs and a couple of other "sensible" places.
It also skips files that are likely to contain meta-code, since there the use of empty lines in definition is more widespread.
This PR continues the work from #25236. |
large-import
maintainer-merge
|
375/5 |
Mathlib.lean,Mathlib/CategoryTheory/Comma/StructuredArrow/CommaMap.lean,Mathlib/Init.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter/EmptyLine.lean,MathlibTest/EmptyLine.lean |
6 |
3 |
['adomani', 'github-actions'] |
nobody |
0-43678 12 hours ago |
14-76295 14 days ago |
14-76350 14 days |
26550 |
Komyyy author:Komyyy |
chore: declare `T₀ ∧ R₀ → T₁` as an instance |
As [instT2SpaceOfR1SpaceOfT0Space](https://leanprover-community.github.io/mathlib4_docs/Mathlib/Topology/Separation/Hausdorff.html#instT2SpaceOfR1SpaceOfT0Space).
I forgot to do this in my PR(#26064).
---
[](https://gitpod.io/from-referrer/)
|
t-topology
easy
|
1/2 |
Mathlib/Topology/Separation/Basic.lean,Mathlib/Topology/Separation/GDelta.lean |
2 |
1 |
['github-actions'] |
nobody |
0-43120 11 hours ago |
0-43120 11 hours ago |
0-43106 11 hours |
26554 |
b-mehta author:b-mehta |
chore(Set/Finite): fix broken link |
---
[](https://gitpod.io/from-referrer/)
|
t-data
easy
documentation
|
1/1 |
Mathlib/Data/Set/Finite/Basic.lean |
1 |
1 |
['github-actions'] |
nobody |
0-40686 11 hours ago |
0-40697 11 hours ago |
0-40743 11 hours |
26366 |
robin-carlier author:robin-carlier |
feat(CategoryTheory/Limits/Shapes/Pullback): categorical pullbacks |
Given a functor `F : A ⥤ B` and `G : C ⥤ B`, `CategoricalPullback F G` is the category of triples `(a : A, c : C, e : F.obj a ≅ G.obj b)`. This construction is to be thought of as an explicit (unbundled) model of the pseudolimit of the cospan in `Cat` defined by `F` and `G`. To justify this claim, after giving some basic API on `CategoricalPullback`, we construct an equivalence of categories between `X ⥤ CategoricalPullback F G` and `CategoricalPullback (whiskeringRight X A B|>.obj F) (whiskeringRight X C B|>.obj G)`, the latter is by definition the categories of triples `(U : X ⥤ A`, `V : X ⥤ C`, `U ⋙ F ≅ V ⋙ G)`, i.e the category of "categorical commutative squares" with top left corner `X` and lying over the cospan defined by `F` and `G`. This equivalence realizes the universal property of the categorical pullback.
This PR is first of a series that aims at bringing API for (2,1)-categorical pullbacks of categories. Further work on the subject includes
* Definition of a type-class extending `CatCommSq _ _ F G` that bundles the assumption that a categorical commutative square is a categorical pullback square, by bundling the data of an equivalence with the categorical pullback of `F` and `G` compatible with the 2-isomorphisms.
* Full 2-functoriality and equivalence-invariance of this notion.
* Horizontal and vertical pasting calculus for categorical pullback squares.
---
- [x] depends on: #26468
[](https://gitpod.io/from-referrer/)
|
t-category-theory |
381/0 |
Mathlib.lean,Mathlib/CategoryTheory/CatCommSq.lean,Mathlib/CategoryTheory/Limits/Shapes/Pullback/Categorical/Basic.lean |
3 |
23 |
['github-actions', 'joelriou', 'mathlib4-dependent-issues-bot', 'robin-carlier'] |
nobody |
0-40425 11 hours ago |
1-27070 1 day ago |
2-24552 2 days |
26521 |
YaelDillies author:YaelDillies |
chore(Algebra/BigOperators): rename variables away from greek letters |
Uniformise the variables to `ι`, `κ` for the indexing types, `M`, `N` for monoids, `G` for groups, `M₀` for monoids with zero, `R` for (semi)rings.
Also delete a duplicated lemma which suddenly became problematic.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
442/456 |
Mathlib/Algebra/BigOperators/Associated.lean,Mathlib/Algebra/BigOperators/Fin.lean,Mathlib/Algebra/BigOperators/Finsupp/Basic.lean,Mathlib/Algebra/BigOperators/Group/Finset/Defs.lean,Mathlib/Algebra/BigOperators/Group/Finset/Lemmas.lean,Mathlib/Algebra/BigOperators/Group/Finset/Piecewise.lean,Mathlib/Algebra/BigOperators/Group/List/Basic.lean,Mathlib/Algebra/BigOperators/Group/List/Lemmas.lean,Mathlib/Algebra/BigOperators/Group/Multiset/Basic.lean,Mathlib/Algebra/BigOperators/Group/Multiset/Defs.lean,Mathlib/Algebra/BigOperators/GroupWithZero/Action.lean,Mathlib/Algebra/BigOperators/Intervals.lean,Mathlib/Algebra/BigOperators/Pi.lean,Mathlib/Algebra/BigOperators/Ring/Finset.lean,Mathlib/Algebra/BigOperators/Ring/Multiset.lean,Mathlib/Algebra/BigOperators/Sym.lean,Mathlib/Algebra/BigOperators/WithTop.lean,Mathlib/Data/Complex/Exponential.lean,Mathlib/FieldTheory/Finite/Polynomial.lean,Mathlib/LinearAlgebra/Matrix/Trace.lean,Mathlib/NumberTheory/LegendreSymbol/JacobiSymbol.lean,Mathlib/NumberTheory/SumPrimeReciprocals.lean |
22 |
7 |
['YaelDillies', 'b-mehta', 'github-actions'] |
nobody |
0-40315 11 hours ago |
0-40315 11 hours ago |
0-40331 11 hours |
26548 |
pechersky author:pechersky |
feat(Algebra/Order/Archimedean): (Mul)Archimedean.comap |
Transferring MulArchimedean across a hom
---
[](https://gitpod.io/from-referrer/)
|
t-order
t-algebra
easy
label:t-algebra$ |
8/0 |
Mathlib/Algebra/Order/Archimedean/Basic.lean |
1 |
1 |
['github-actions'] |
nobody |
0-39747 11 hours ago |
0-45838 12 hours ago |
0-45840 12 hours |
26507 |
MichaelStollBayreuth author:MichaelStollBayreuth |
feat(Algebra/Polynomial/Degree/IsMonicOfDegree): new file |
This adds a predicate `Polynomial.IsMonicOfDegree p n` expressing that the polynomial `p` is monic and has `natDegree` equal to `n` and provides some API for it.
Bundling the two properties is quite convenient (e.g., showing that the product of two monic polynomials of degrees `m` and `n` is monic of degree `m+n` needs a few lines with the currently available API) and proved very helpful for formalizing a proof of the Gelfand-Mazur theorem over the reals.
See also here on Zulip : [#mathlib4 > Gelfand-Mazur theorem @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Gelfand-Mazur.20theorem/near/525404185).
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
276/0 |
Mathlib.lean,Mathlib/Algebra/Polynomial/Degree/IsMonicOfDegree.lean |
2 |
10 |
['MichaelStollBayreuth', 'adomani', 'github-actions'] |
riccardobrasca assignee:riccardobrasca |
0-37761 10 hours ago |
1-61791 1 day ago |
1-61776 1 day |
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 |
0-35971 9 hours ago |
12-43221 12 days ago |
12-43226 12 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 `mapM 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.fold`, `FreeWriter.fold`, `FreeCont.fold`) derived from
the universal property via `mapM`
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
|
717/0 |
Mathlib.lean,Mathlib/Control/Monad/Free.lean,MathlibTest/freemonad.lean,docs/references.bib |
4 |
144 |
['YaelDillies', 'copilot-pull-request-reviewer', 'eric-wieser', 'github-actions', 'plp127', 'quangvdao', 'tannerduve'] |
nobody |
0-35534 9 hours ago |
13-48251 13 days ago |
23-67335 23 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.
- [ ] depends on #25949
---
[](https://gitpod.io/from-referrer/)
|
new-contributor |
117/0 |
Mathlib.lean,Mathlib/Analysis/InnerProductSpace/MulOpposite.lean,Mathlib/LinearAlgebra/Basis/MulOpposite.lean |
3 |
1 |
['github-actions'] |
nobody |
0-34240 9 hours ago |
14-64463 14 days ago |
14-64456 14 days |
26556 |
fweth author:fweth |
feat(CategoryTheory/Topos): subobject classifier without limits |
Adds an alternative API for constructing a subobject classifier without reference to limits.
This PR modifies two files:
* `Mathlib/CategoryTheory/Limits/Shapes/Pullback/CommSq.lean`:
Adds strengthened versions of two existing theorems:
- `of_horiz_isIso_mono` (alongside the existing `of_horiz_isIso`)
- `of_vert_isIso_mono` (alongside the existing `of_vert_isIso`)
* `Mathlib/CategoryTheory/Topos/Classifier.lean`:
Addresses the TODO (removed from the file):
> Make API for constructing a subobject classifier without reference to limits (replacing `⊤_ C` with an arbitrary `Ω₀ : C` and including the assumption `mono truth`)
This implementation assumes a monomorphism `truth : Ω₀ ⟶ Ω` such that for each monomorphism `m : U ⟶ X` there exists a unique pair `χ₀ : U ⟶ Ω₀` and `χ : X ⟶ Ω` which create a pullback square. Given these ingrediences, we construct an instance of the existing `Classifier` structure, alongside with a proof that `Ω₀` is terminal. Other interpretations of the TODO are possible, feel free to request a different one.
Klaus Gy
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-category-theory
|
81/6 |
Mathlib/CategoryTheory/Limits/Shapes/Pullback/CommSq.lean,Mathlib/CategoryTheory/Topos/Classifier.lean |
2 |
1 |
['github-actions'] |
nobody |
0-31751 8 hours ago |
0-33838 9 hours ago |
0-33883 9 hours |
26557 |
b-mehta author:b-mehta |
feat(ENNReal): add div_div_cancel |
Two new lemmas, with names matching their group versions.
---
[](https://gitpod.io/from-referrer/)
|
t-data
easy
|
15/0 |
Mathlib/Data/ENNReal/Inv.lean |
1 |
1 |
['github-actions'] |
nobody |
0-31611 8 hours ago |
0-31618 8 hours ago |
0-31666 8 hours |
26336 |
mans0954 author:mans0954 |
feat(Topology/Order/HullKernel): Add the Hull-Kernel Topology |
Let `α` be a `CompleteLattice` and let `T` be a subset of `α`. The relative `Topology.lower` on `T`
takes on a particularly simple form when every element of `T` is `InfPrime` in `α`. In this case,
the relative-open sets are exactly the sets of the form `T ↓∩ (Ici a)ᶜ` for some `a` in `α`.
The pair of maps `S → ⊓ S` and `a → T ↓∩ Ici a` are often referred to as the kernel and the hull.
They form an antitone Galois connection between the subsets of `T` and `α`. When `α` can be generated
from `T` by taking infs, this becomes a Galois insertion and the topological closure coincides with
the closure arising from the Galois insertion. For this reason the relative lower topology on `T` is
often referred to as the "hull-kernel topology". The names "Jacobson topology" and "structure topology"
also occur in the literature.
---
This PR continues the work from #13918.
Original PR: https://github.com/leanprover-community/mathlib4/pull/13918
[](https://gitpod.io/from-referrer/) |
t-topology |
272/0 |
Mathlib.lean,Mathlib/Topology/Order/HullKernel.lean,docs/references.bib |
3 |
n/a |
['YaelDillies', 'github-actions', 'mans0954'] |
nobody |
0-31492 8 hours ago |
unknown |
unknown |
26505 |
sgouezel author:sgouezel |
feat: in a continuous Riemannian bundle, the trivialization at a point is locally bounded in norm |
This follows from the continuity of the bilinear form defining the norm, although the reduction requires some care.
---
[](https://gitpod.io/from-referrer/)
|
t-topology |
275/1 |
Mathlib/Topology/VectorBundle/Constructions.lean,Mathlib/Topology/VectorBundle/Hom.lean,Mathlib/Topology/VectorBundle/Riemannian.lean |
3 |
4 |
['github-actions', 'grunweg', 'sgouezel'] |
nobody |
0-29596 8 hours ago |
1-81996 1 day ago |
1-81980 1 day |
26543 |
vihdzp author:vihdzp |
feat(SetTheory/ZFC/VonNeumann): von Neumann hierarchy of sets |
Ported from #17027. For extra discussion on this PR, see [Zulip](https://leanprover.zulipchat.com/#narrow/channel/144837-PR-reviews/topic/.2317027.20.2C.20.2326518.20von.20Neumann.20hierarchy/with/526389347).
---
[](https://gitpod.io/from-referrer/)
|
t-set-theory
maintainer-merge
|
133/0 |
Mathlib.lean,Mathlib/SetTheory/Ordinal/Basic.lean,Mathlib/SetTheory/ZFC/Basic.lean,Mathlib/SetTheory/ZFC/VonNeumann.lean |
4 |
55 |
['alreadydone', 'github-actions', 'kckennylau', 'vihdzp'] |
nobody |
0-24644 6 hours ago |
0-24885 6 hours ago |
0-54425 15 hours |
25910 |
themathqueen author:themathqueen |
feat(Algebra/Ring/Idempotent): for idempotent `p,q`, `q-p` is idempotent iff `pq=p=qp` |
Added useful lemmas for idempotents and projections.
Main result:
- IsIdempotentElem.sub_iff: if `p` and `q` are idempotent elements, then `q - p` is idempotent iff `p * q = p = q * p`
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-algebra
label:t-algebra$ |
89/0 |
Mathlib/Algebra/Ring/Idempotent.lean,Mathlib/LinearAlgebra/Projection.lean |
2 |
23 |
['github-actions', 'tb65536', 'themathqueen'] |
nobody |
0-22393 6 hours ago |
0-82450 22 hours ago |
3-30213 3 days |
26533 |
winstonyin author:winstonyin |
feat: fix definition of `IsIntegralCurveOn` for consistency |
I change the definition of `IsIntegralCurveOn` to use `HasMFDerivWithinAt`, rather than `HasMFDerivAt`, so as to make this definition consistent with `DifferentiableOn` and `ContinuousOn`. While the API around it slightly changes, there is no effect on the statement of any downstream lemmas.
---
[](https://gitpod.io/from-referrer/)
|
maintainer-merge
t-differential-geometry
|
89/58 |
Mathlib/Geometry/Manifold/IntegralCurve/Basic.lean,Mathlib/Geometry/Manifold/IntegralCurve/ExistUnique.lean,Mathlib/Geometry/Manifold/IntegralCurve/Transform.lean,Mathlib/Geometry/Manifold/IntegralCurve/UniformTime.lean |
4 |
14 |
['github-actions', 'grunweg', 'winstonyin'] |
grunweg assignee:grunweg |
0-17799 4 hours ago |
0-24256 6 hours ago |
0-57779 16 hours |
26404 |
grunweg author:grunweg |
chore: clean up and remove FunProp/Differentiable |
- one lemma in that file already exists, hence can be removed
(We don't add a deprecation as I presume people will not have used it.)
- move the three remaining lemmas in that file to their proper place, and use the now `fun_` naming convention
(Omitting deprecations again.)
- after this, `FunProp/Differentiable` is empty and need not be imported any more: add a module deprecation
---
- [x] depends on: #26355
[](https://gitpod.io/from-referrer/)
|
tech debt |
23/49 |
Mathlib/Analysis/Calculus/FDeriv/Comp.lean,Mathlib/Tactic/FunProp/ContDiff.lean,Mathlib/Tactic/FunProp/Differentiable.lean,MathlibTest/fun_prop2.lean |
4 |
3 |
['github-actions', 'grunweg', 'mathlib4-dependent-issues-bot'] |
nobody |
0-17793 4 hours ago |
5-43559 5 days ago |
5-43605 5 days |
25872 |
101damnations author:101damnations |
feat(RepresentationTheory/GroupCohomology): long exact sequences |
Given a commutative ring `k` and a group `G`, this PR shows that a short exact sequence of `k`-linear `G`-representations
`0 ⟶ X₁ ⟶ X₂ ⟶ X₃ ⟶ 0` induces a short exact sequence of complexes `0 ⟶ C(X₁) ⟶ C(X₂) ⟶ C(X₃) ⟶ 0`, where `C(Xᵢ)` is the complex of inhomogeneous cochains of `Xᵢ`, and hence `Hⁿ(C(Xᵢ))` is the `n`th group cohomology of `Xᵢ`.
---
- [x] depends on: #25815
- [x] depends on: #25870
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #25311.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/25311*
|
maintainer-merge
t-algebra
label:t-algebra$ |
289/7 |
Mathlib.lean,Mathlib/Algebra/Homology/ConcreteCategory.lean,Mathlib/Algebra/Homology/HomologySequence.lean,Mathlib/Algebra/Homology/ShortComplex/SnakeLemma.lean,Mathlib/LinearAlgebra/Pi.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/Basic.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/LongExactSequence.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/LowDegree.lean |
8 |
9 |
['101damnations', 'github-actions', 'kbuzzard', 'mathlib4-dependent-issues-bot'] |
nobody |
0-16826 4 hours ago |
1-22683 1 day ago |
14-3080 14 days |
26560 |
b-mehta author:b-mehta |
chore(Topology/LiminfLimsup): split out non-algebraic content from Topology/Algebra file |
All the moved content had no algebraic material (in particular required no algebraic imports), so we move it out of Topology/Algebra. This increases discoverability and improves the global organisation of `Topology/`, and gives a net import decrease across mathlib.
---
[](https://gitpod.io/from-referrer/)
|
t-topology |
411/382 |
Mathlib.lean,Mathlib/Analysis/Asymptotics/Lemmas.lean,Mathlib/Analysis/Normed/Group/Ultra.lean,Mathlib/Analysis/Normed/Lp/lpSpace.lean,Mathlib/Analysis/Normed/Unbundled/SmoothingSeminorm.lean,Mathlib/MeasureTheory/Integral/BoundedContinuousFunction.lean,Mathlib/Order/Filter/ENNReal.lean,Mathlib/Topology/Algebra/Order/LiminfLimsup.lean,Mathlib/Topology/Instances/ENNReal/Lemmas.lean,Mathlib/Topology/Order/LiminfLimsup.lean |
10 |
1 |
['github-actions'] |
nobody |
0-16370 4 hours ago |
0-29760 8 hours ago |
0-29829 8 hours |
26513 |
wwylele author:wwylele |
feat(Order): complementary under sublattice |
This makes the `complementedLattice_Iic` instance more discoverable by stating
the theorem that `ComplementedLattice` + `ModularLattice` -> one can find a complement
relative to any pair of elements.
---
~~While the proof is short from order theory perspective, there wasn't an obvious theorem stating that you can also take complementary submodule under a larger submodule. Add this here for better discovery.~~
[](https://gitpod.io/from-referrer/)
|
t-algebra
easy
label:t-algebra$ |
35/30 |
Mathlib/Order/ModularLattice.lean |
1 |
15 |
['eric-wieser', 'github-actions', 'wwylele'] |
nobody |
0-14570 4 hours ago |
1-45955 1 day ago |
1-46005 1 day |
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 |
0-13431 3 hours ago |
14-64258 14 days ago |
14-72861 14 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`.
---
- [x] depends on: #9951
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-meta
label:t-algebra$ |
732/211 |
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/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/ring.lean |
17 |
6 |
['eric-wieser', 'github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'plp127'] |
nobody |
0-11610 3 hours ago |
3-38995 3 days ago |
3-38987 3 days |
26552 |
Komyyy author:Komyyy |
feat: equivalent condition for subgroups to be simple |
And simpleness of isomorphic groups are equivalent.
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$ |
23/1 |
Mathlib/GroupTheory/Subgroup/Simple.lean |
1 |
1 |
['github-actions'] |
nobody |
0-7766 2 hours ago |
0-41791 11 hours ago |
0-41777 11 hours |
26555 |
Komyyy author:Komyyy |
feat: lemmas about betweeness on a linear space |
This PR also adds aliases of the inverse direction of betweeness iff lemmas.
---
[](https://gitpod.io/from-referrer/)
|
t-euclidean-geometry |
86/0 |
Mathlib/Analysis/Convex/Between.lean |
1 |
1 |
['github-actions'] |
nobody |
0-7667 2 hours ago |
0-35662 9 hours ago |
0-38872 10 hours |
26392 |
winstonyin author:winstonyin |
feat: solution to ODE is Lipschitz with respect to the initial condition |
This PR continues the work from #20733.
Original PR: https://github.com/leanprover-community/mathlib4/pull/20733
I formalise a corollary to the Picard-Lindelöf theorem: the local solution to an ODE is Lipschitz continuous with respect to the initial condition. This in particular means that the local flow to the associated vector field is continuous.
- [ ] depends on: #26382
---
[](https://gitpod.io/from-referrer/)
|
t-dynamics
t-analysis
|
127/1 |
Mathlib/Analysis/ODE/PicardLindelof.lean |
1 |
10 |
['AntoineChambert-Loir', 'github-actions', 'grunweg', 'mathlib4-dependent-issues-bot', 'winstonyin'] |
nobody |
0-5644 1 hour ago |
0-53254 14 hours ago |
0-54317 15 hours |
26538 |
mariainesdff author:mariainesdff |
feat(RingTheory/Valuation/Extension): add algebra instances |
Provide algebra instances for valuation subrings and residue fields.
Co-authored-by: @faenuccio
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebra
label:t-algebra$ |
57/4 |
Mathlib/RingTheory/Valuation/Extension.lean |
1 |
7 |
['github-actions', 'mariainesdff', 'pechersky'] |
nobody |
0-5630 1 hour ago |
0-65621 18 hours ago |
0-65669 18 hours |