Welcome to the PR triage page! This page is perfect if you intend to look for pull request which seem to have stalled.
Feedback on designing this page or further information to include is very welcome.
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 |
14444 |
digama0 author:digama0 |
fix(GeneralizeProofs): unreachable! bug |
As [reported on Zulip](https://leanprover.zulipchat.com/#narrow/stream/270676-lean4/topic/Unreachable.20code.20reached.20in.20Lean.204.2E8.2E0/near/449286780).
---
[](https://gitpod.io/from-referrer/)
|
t-meta
awaiting-author
|
1/1 |
Mathlib/Tactic/GeneralizeProofs.lean |
1 |
4 |
['github-actions', 'jcommelin', 'kmill'] |
nobody |
409-8944 1 year ago |
424-46514 1 year ago |
10-36842 10 days |
14345 |
digama0 author:digama0 |
feat: the Dialectica category is monoidal closed |
- [x] depends on: #14274
The monoidal closed structure of the Dialectica category.
---
[](https://gitpod.io/from-referrer/)
|
t-category-theory
awaiting-author
|
252/0 |
Mathlib.lean,Mathlib/CategoryTheory/Dialectica/Closed.lean |
2 |
3 |
['github-actions', 'kim-em', 'leanprover-community-mathlib4-bot'] |
nobody |
409-8944 1 year ago |
424-63348 1 year ago |
12-17890 12 days |
12952 |
adomani author:adomani |
test: length statistics |
---
[](https://gitpod.io/from-referrer/)
|
test-ci
WIP
|
124/0 |
.github/workflows/mathlib_stats.yml,.github/workflows/ml_stats_label.yaml,scripts/mathlib_stats.sh |
3 |
9 |
['github-actions'] |
nobody |
409-8943 1 year ago |
437-68023 1 year ago |
0-0 0 seconds |
12452 |
JADekker author:JADekker |
feat(Cocardinal) : add some more api |
Just a small PR to add a bit more API for cocardinal filters. Not everything seems to generalise nicely from cofinite, so I didn't include such results.
Currently the file has one `sorry`, I'm not sure how to complete this proof.
---
[](https://gitpod.io/from-referrer/)
|
t-topology
awaiting-CI
|
75/0 |
Mathlib/Order/Filter/Cocardinal.lean |
1 |
0 |
[] |
nobody |
409-8942 1 year ago |
430-76042 1 year ago |
0-0 0 seconds |
12984 |
adomani author:adomani |
Adomani/periodic reports dev custom action |
---
[](https://gitpod.io/from-referrer/)
|
test-ci
WIP
|
366/0 |
.github/workflows/mathlib_stats.yml,.github/workflows/ml_stats_label.yaml,scripts/count_decls.lean,scripts/mathlib_stats.sh |
4 |
n/a |
['github-actions'] |
nobody |
409-8942 1 year ago |
unknown |
unknown |
11991 |
adomani author:adomani |
draft: syntax data linter |
A linter that prints `SyntaxNodeKind`s and `Range`s for all the nodes of a command.
See this [Zulip discussion](https://leanprover.zulipchat.com/#narrow/stream/217875-Is-there-code-for-X.3F/topic/undocumented.20things).
---
[](https://gitpod.io/from-referrer/)
|
WIP |
152/0 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/SyntaxDataLinter.lean |
3 |
0 |
[] |
nobody |
409-8941 1 year ago |
437-68016 1 year ago |
0-0 0 seconds |
10099 |
mcdoll author:mcdoll |
feat: Integration by parts for higher dimensional spaces |
---
- [x] depends on: #9987
- [x] depends on: #10105
- [x] depends on: #10107
- [x] depends on: #10115
- [x] depends on: #10118
- [x] depends on: #10182
[](https://gitpod.io/from-referrer/)
|
t-measure-probability
t-analysis
WIP
|
429/0 |
Mathlib/Analysis/InnerProductSpace/OrthoDecomp.lean,Mathlib/MeasureTheory/Integral/test2.lean |
2 |
3 |
['alexjbest', 'github-actions', 'leanprover-community-mathlib4-bot'] |
nobody |
409-8940 1 year ago |
582-39357 1 year ago |
0-0 0 seconds |
10998 |
hmonroe author:hmonroe |
feat(Logic): Arithmetization of partial recursive functions (toward Gödel's first incompleteness theorem) |
---
[](https://gitpod.io/from-referrer/)
|
t-logic
awaiting-author
|
364/0 |
Mathlib.lean,Mathlib/Logic/Godel/PartArith.lean |
2 |
3 |
['Ruben-VandeVelde', 'YaelDillies'] |
nobody |
409-8940 1 year ago |
463-66576 1 year ago |
97-20483 97 days |
9469 |
dupuisf author:dupuisf |
feat: maximum modulus principle for functions vanishing at infinity |
This PR adds versions of the maximum modulus principle for functions vanishing at infinity that parallel those we already had for functions over a bounded set. These will have applications in e.g. norm interpolation.
---
[](https://gitpod.io/from-referrer/)
|
t-analysis
awaiting-author
|
71/0 |
Mathlib/Analysis/Complex/AbsMax.lean |
1 |
8 |
['dupuisf', 'j-loreaux'] |
nobody |
409-8939 1 year ago |
603-50185 1 year ago |
12-86009 12 days |
9510 |
eric-wieser author:eric-wieser |
feat(Analysis/Calculus/DualNumber): Extending differentiable functions to dual numbers |
This shows that this operation preserves multiplication and composition
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-analysis
awaiting-CI
WIP
label:t-algebra$ |
119/0 |
Mathlib/Analysis/Calculus/DualNumber.lean |
1 |
4 |
['github-actions'] |
nobody |
409-8939 1 year ago |
614-83370 1 year ago |
0-0 0 seconds |
9352 |
chenyili0818 author:chenyili0818 |
feat: arithmetic lemmas for `gradient` |
This file is based on Mathlib.Analysis.Calculus.Gradient.Basic, and describes the calculation properties
Co-authored-by: Ziyu Wang [tropicalfish910@gmail.com](mailto:tropicalfish910@gmail.com)
---
[](https://gitpod.io/from-referrer/)
|
t-analysis
awaiting-author
|
404/0 |
Mathlib.lean,Mathlib/Analysis/Calculus/Gradient/Lemmas.lean |
2 |
30 |
['chenyili0818', 'github-actions', 'jcommelin', 'sgouezel', 'winstonyin'] |
nobody |
409-8939 1 year ago |
570-76504 1 year ago |
51-80670 51 days |
6859 |
MohanadAhmed author:MohanadAhmed |
TryLean4Bundle: Windows Bundle Creator |
# `TryLean4Bundle`: Windows Bundle Creator
A Windows batch script and a CI yml file that create an self extracting archive. The user should
1. just download the archive,
2. double click the archive to expand
3. double click the `RunLean.bat` script in the expanded archive.
The script currently downloads 7 dependencies into CI then unpacks them in the appropriate locations and finally packs them back.
To try a bundle created using these scripts but from a different repo see (https://github.com/MohanadAhmed/TryLean4Bundle/releases)
---
[](https://gitpod.io/from-referrer/)
|
CI
WIP
help-wanted
|
114/0 |
.github/workflows/mk_windows_bundle.yml,scripts/windowsBundle.bat |
2 |
0 |
[] |
nobody |
409-8938 1 year ago |
745-38209 2 years ago |
0-0 0 seconds |
7125 |
eric-wieser author:eric-wieser |
feat: additive monoid structure via biproducts |
I suspect I'm missing a trick with these transport lemmas.
---
[](https://gitpod.io/from-referrer/)
|
t-category-theory
awaiting-CI
WIP
|
237/0 |
Mathlib/CategoryTheory/Limits/Skeleton.lean |
1 |
2 |
['alreadydone', 'eric-wieser'] |
nobody |
409-8938 1 year ago |
718-83079 1 year ago |
0-0 0 seconds |
7890 |
grhkm21 author:grhkm21 |
feat(Mathlib/Tactic/Setm): implement setm tactic |
This is my first time doing metaprogramming in Lean 4, please provide feedback when you have them :)
The `setm` tactic, which stands for `set` + matching, matches a given expression with the goal and introduces new local hypotheses for the named holes specified. One of the best usage is for rearrangement proofs. As a simple example,
```lean
example : (1 + 1) + (4 * 3) - (1 + 1) = (3 * 4 : Rat) := by
setm ?A + ?B - ?A = (?C : Rat)
rw [show ∀ A B, A + B - A = B by intro A B ; ring_nf ]
apply Rat.mul_comm
```
One can imagine replacing the three term expression with a 7 term algebraic expression.
This was developed with tons of help from [Zulip](https://leanprover.zulipchat.com/#narrow/stream/239415-metaprogramming-.2F-tactics/topic/Help.20with.20writing.20tactic), especially from Thomas. Thanks!
TODO:
- [X] Support `setm ... at ...` syntax, see *example 1* below
- [X] Write docs
- [ ] Use `withNewMCtxDepth`
- [X] Rename the intermediate `MVar`s, see *example 2* below
- [ ] Use `elabTermWithHolesPostponing` in conjunction with `Term.synthesizeSyntheticMVarsNoPostPoning` after `isDefEq` to handle instances
Example 1:
```lean
/- Usage with `using` and `at` keywords -/
example (h1 : 1 + 1 = 3) (h2 : 1 + 3 = 5) (h3 : 2 + 2 = 5) : true := by
setm ?A + _ = (?B : Nat) using h2 at h1 h2 h3
guard_hyp A := 1
guard_hyp B := 5
guard_hyp h1 : A + A = 3
guard_hyp h2 : A + 3 = B
guard_hyp h3 : 2 + 2 = B
trivial
```
Example 2:
```lean
/- Test reusing named holes -/
example (h : b + a = c) : a + b = c := by
/- setm 1-/
setm ?A + ?B = (_ : Nat)
guard_hyp A := a
guard_hyp B := b
/- clean up -/
unfold_let A B
clear hA hB A B
/- setm 2 -/
rewrite [Nat.add_comm]
setm ?A + ?B = (_ : Nat) at h ⊢
guard_hyp A := b
guard_hyp B := a
exact h
```
Co-authored-by: Jireh Loreaux
[](https://gitpod.io/from-referrer/)
|
t-meta |
141/0 |
Mathlib.lean,Mathlib/Tactic/Common.lean,Mathlib/Tactic/Setm.lean,test/Setm.lean |
4 |
3 |
['thorimur'] |
nobody |
409-8938 1 year ago |
690-10462 1 year ago |
0-0 0 seconds |
8224 |
Kha author:Kha |
chore: add `lean4checker` benchmark |
|
WIP |
16/0 |
scripts/bench/temci-config.run.yml |
1 |
3 |
['Kha', 'grunweg', 'kim-em', 'leanprover-bot'] |
nobody |
409-8938 1 year ago |
476-61867 1 year ago |
0-0 0 seconds |
5745 |
alexjbest author:alexjbest |
feat: a tactic to consume type annotations, and make constructor nicer |
During the copenhagen masterclass I found some situations where applying the constructor tactic left the goal in a difficult to read state when autoParams were present.
We add a simple tactic to clean these up, and a macro for `constructor` to behave more like the constructor notation and do this automatically (constructor is in core)
It seems that these things should be cleaned up by simp, but a simp lemma to remove these annotations is not accepted by lean as the types are too similar.
---
[](https://gitpod.io/from-referrer/)
|
t-meta
awaiting-author
|
41/0 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Consume.lean,test/consume.lean |
4 |
4 |
['alexjbest', 'digama0', 'kim-em', 'kmill'] |
nobody |
409-8937 1 year ago |
493-58831 1 year ago |
51-33797 51 days |
4786 |
thorimur author:thorimur |
feat: AppBuilder utils |
This supplements `Lean.Meta.AppBuilder`, introducing variants of `mkAppN` and `mkAppM` which allow for more fine-grained management of existing and created metavariables. [Description pending]
---
[](https://gitpod.io/from-referrer/)
|
t-meta |
205/0 |
Mathlib.lean,Mathlib/Lean/Meta/AppBuilder.lean |
2 |
0 |
[] |
nobody |
409-8937 1 year ago |
829-9291 2 years ago |
0-0 0 seconds |
15224 |
AnthonyBordg author:AnthonyBordg |
feat(CategoryTheory/Sites): covering families and their associated Grothendieck topology |
Define covering families on a category and their associated Grothendieck topology by using the API for `Coverage`.
Give an explicit characterization of the covering sieves of the said topology.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-category-theory
awaiting-author
|
112/0 |
Mathlib.lean,Mathlib/CategoryTheory/Sites/CoveringFamilies.lean |
2 |
20 |
['AnthonyBordg', 'adamtopaz', 'dagurtomas', 'github-actions', 'joelriou'] |
nobody |
403-70354 1 year ago |
408-64019 1 year ago |
1-48443 1 day |
15453 |
tomaz1502 author:tomaz1502 |
Track formalization of runtime complexity |
I finished porting https://github.com/leanprover-community/mathlib3/pull/14494/ to Lean 4 and made several small PRs, as suggested. This meta PR is used to track the progress of the smaller PRs.
## Pending PRs
- [Formalization of List.insertionSort](https://github.com/leanprover-community/mathlib4/pull/15449)
- [Lemmas about Split](https://github.com/leanprover-community/mathlib4/pull/15450)
- [Formalization of List.merge](https://github.com/leanprover-community/mathlib4/pull/15451)
- [Formalization of List.mergeSort](https://github.com/leanprover-community/mathlib4/pull/15452)
---
[](https://gitpod.io/from-referrer/)
|
|
525/0 |
Mathlib.lean,Mathlib/Computability/Timed/InsertionSort.lean,Mathlib/Computability/Timed/Merge.lean,Mathlib/Computability/Timed/MergeSort.lean,Mathlib/Computability/Timed/Split.lean |
5 |
4 |
['joneugster', 'mergify'] |
nobody |
395-3222 1 year ago |
395-3276 1 year ago |
0-0 0 seconds |
14563 |
awueth author:awueth |
feat: if-then-else of exclusive or statement |
---
If `¬(P ∧ Q)` then `ite (P ∨ Q) a 1 = (ite P a 1) * (ite Q a 1)`
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-algebra
awaiting-author
label:t-algebra$ |
5/0 |
Mathlib/Algebra/Group/Basic.lean |
1 |
3 |
['eric-wieser', 'github-actions', 'kim-em'] |
nobody |
394-1330 1 year ago |
394-1330 1 year ago |
6-38745 6 days |
10387 |
adomani author:adomani |
feat(Tactic/ComputeDegree): add `polynomial` tactic |
Introducing the `polynomial` tactic, summing up `compute_degree, monicity` and adding support for `leadingCoeff`.
This is more of a proof of concept: if there is interest in this tactic, I can polish it up.
See [this Zulip discussion](https://leanprover.zulipchat.com/#narrow/stream/113489-new-members/topic/Compute.20roots.20of.20polynomials/near/420713624).
---
[](https://gitpod.io/from-referrer/)
|
RFC
t-meta
WIP
|
24/0 |
Mathlib/Tactic/ComputeDegree.lean |
1 |
0 |
[] |
nobody |
393-84878 1 year ago |
393-84878 1 year ago |
0-0 0 seconds |
9693 |
madvorak author:madvorak |
feat: Linear programming in the standard form |
---
Zulip discussion:
https://leanprover.zulipchat.com/#narrow/stream/144837-PR-reviews/topic/.237386.20Linear.20Programming
Four PRs incompatible with each other:
https://github.com/leanprover-community/mathlib4/pull/7386 (list of constraints)
https://github.com/leanprover-community/mathlib4/pull/9693 (matrix form)
https://github.com/leanprover-community/mathlib4/pull/10026 (Antoine Chambert-Loir's def; semirings, linear)
https://github.com/leanprover-community/mathlib4/pull/10159 (Antoine Chambert-Loir's def; rings, affine)
- [x] depends on: #9652
[](https://gitpod.io/from-referrer/)
|
t-algebra
RFC
WIP
label:t-algebra$ |
86/0 |
Mathlib.lean,Mathlib/LinearAlgebra/Matrix/LinearProgramming.lean |
2 |
14 |
['apurvanakade', 'github-actions', 'leanprover-community-mathlib4-bot', 'madvorak'] |
nobody |
393-84793 1 year ago |
393-84793 1 year ago |
0-0 0 seconds |
7386 |
madvorak author:madvorak |
feat: Define linear programs |
Linear programs over a general `Module` with constraints given in the form "aᵀx - b ≥ 0" and the objective function as an `AffineMap` to be minimized.
---
Zulip discussion:
https://leanprover.zulipchat.com/#narrow/stream/144837-PR-reviews/topic/.237386.20Linear.20Programming
Four PRs incompatible with each other:
https://github.com/leanprover-community/mathlib4/pull/7386 (list of constraints)
https://github.com/leanprover-community/mathlib4/pull/9693 (matrix form)
https://github.com/leanprover-community/mathlib4/pull/10026 (Antoine Chambert-Loir's def; semirings, linear)
https://github.com/leanprover-community/mathlib4/pull/10159 (Antoine Chambert-Loir's def; rings, affine)
[](https://gitpod.io/from-referrer/)
|
t-algebra
RFC
WIP
label:t-algebra$ |
87/0 |
Mathlib.lean,Mathlib/LinearAlgebra/LinearProgramming.lean |
2 |
63 |
['Shreyas4991', 'YaelDillies', 'eric-wieser', 'github-actions', 'kim-em', 'madvorak'] |
nobody |
393-84403 1 year ago |
393-84403 1 year ago |
66-6720 66 days |
7219 |
Ruben-VandeVelde author:Ruben-VandeVelde |
feat: Equivs for AddMonoidAlgebras |
---
Extracted from #6718.
[](https://gitpod.io/from-referrer/)
|
t-algebra
awaiting-author
label:t-algebra$ |
113/0 |
Mathlib.lean,Mathlib/Algebra/MonoidAlgebra/Equiv.lean |
2 |
12 |
['Ruben-VandeVelde', 'alreadydone', 'eric-wieser'] |
eric-wieser assignee:eric-wieser |
393-84365 1 year ago |
393-84366 1 year ago |
0-0 0 seconds |
13163 |
erdOne author:erdOne |
feat(.vscode/module-docstring.code-snippet): Prevent auto-complete from firing on `do` |
---
[](https://gitpod.io/from-referrer/)
|
t-meta
awaiting-author
|
5/0 |
.vscode/module-docstring.code-snippets |
1 |
5 |
['erdOne', 'grunweg', 'robertylewis', 'trivial1711'] |
nobody |
393-83192 1 year ago |
393-83192 1 year ago |
50-50444 50 days |
10026 |
madvorak author:madvorak |
Linear programming according to Antoine Chambert-Loir's book |
---
Zulip discussion:
https://leanprover.zulipchat.com/#narrow/stream/144837-PR-reviews/topic/.237386.20Linear.20Programming
Four PRs incompatible with each other:
https://github.com/leanprover-community/mathlib4/pull/7386 (list of constraints)
https://github.com/leanprover-community/mathlib4/pull/9693 (matrix form)
https://github.com/leanprover-community/mathlib4/pull/10026 (Antoine Chambert-Loir's def; semirings, linear)
https://github.com/leanprover-community/mathlib4/pull/10159 (Antoine Chambert-Loir's def; rings, affine)
[](https://gitpod.io/from-referrer/)
|
t-algebra
RFC
WIP
label:t-algebra$ |
86/0 |
Mathlib.lean,Mathlib/LinearAlgebra/LinearProgramming.lean |
2 |
9 |
['eric-wieser', 'madvorak', 'riccardobrasca'] |
nobody |
392-62256 1 year ago |
392-62256 1 year ago |
0-0 0 seconds |
10159 |
madvorak author:madvorak |
Linear programming according to Antoine Chambert-Loir's book — affine version |
---
Zulip discussion:
https://leanprover.zulipchat.com/#narrow/stream/144837-PR-reviews/topic/.237386.20Linear.20Programming
Four PRs incompatible with each other:
https://github.com/leanprover-community/mathlib4/pull/7386 (list of constraints)
https://github.com/leanprover-community/mathlib4/pull/9693 (matrix form)
https://github.com/leanprover-community/mathlib4/pull/10026 (Antoine Chambert-Loir's def; semirings, linear)
https://github.com/leanprover-community/mathlib4/pull/10159 (Antoine Chambert-Loir's def; rings, affine)
[](https://gitpod.io/from-referrer/)
|
t-algebra
RFC
WIP
label:t-algebra$ |
83/0 |
Mathlib.lean,Mathlib/LinearAlgebra/LinearProgramming.lean |
2 |
7 |
['eric-wieser', 'madvorak', 'riccardobrasca'] |
nobody |
392-62242 1 year ago |
392-62242 1 year ago |
0-0 0 seconds |
11890 |
adomani author:adomani |
feat: the terminal refine linter |
A linter that warns on usages of `refine` and `refine'` as a finishing tactic.
See this [Zulip discussion](https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/Usage.20of.20refine').
### Conclusion of the experiment
Systematic replacements of terminal `refine` with `exact` leads to an overall slow-down.
---
- [ ] depends on: #15616 (disable the linter in downstream projects)
[](https://gitpod.io/from-referrer/)
|
t-linter
awaiting-author
|
77/0 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter/TerminalRefineLinter.lean |
3 |
14 |
['adomani', 'github-actions', 'grunweg', 'joneugster', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'urkud'] |
nobody |
390-9423 1 year ago |
390-9425 1 year ago |
18-13508 18 days |
11207 |
luigi-massacci author:luigi-massacci |
feat(Topology/MetricSpace): Add new file with type of Katetov maps |
add a type of Katetov maps (one point extensions of a metric) and related notation and FunLike coercions.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-topology
WIP
|
138/0 |
Mathlib.lean,Mathlib/Topology/MetricSpace/Katetov.lean,docs/references.bib |
3 |
16 |
['fpvandoorn', 'jcommelin', 'kim-em', 'luigi-massacci', 'urkud'] |
nobody |
389-72107 1 year ago |
491-74192 1 year ago |
26-83567 26 days |
11090 |
pangelinos author:pangelinos |
feat: define spectral spaces and prove that a quasi-compact open of a spectral space is spectral |
Define spectral spaces and prove that a quasi-compact open of a spectral space is spectral.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-topology
please-adopt
good first issue
|
69/0 |
Topology/Spectral/basic.lean |
1 |
15 |
['YaelDillies', 'adomani', 'j-loreaux', 'jcommelin', 'kim-em', 'pangelinos'] |
nobody |
389-71982 1 year ago |
393-84908 1 year ago |
16-44803 16 days |
9795 |
sinhp author:sinhp |
feat: the type `Fib` of fibre of a function at a point |
This is the most basic file of the theory of fibred categories developed here: https://github.com/sinhp/LeanFibredCategories/tree/master
---
[](https://gitpod.io/from-referrer/)
|
t-category-theory
awaiting-author
|
74/0 |
Mathlib.lean,Mathlib/Data/Fiber.lean |
2 |
17 |
['adri326', 'joelriou', 'sinhp'] |
nobody |
387-74758 1 year ago |
603-7825 1 year ago |
1-32924 1 day |
15055 |
sinhp author:sinhp |
feat: the category of pointed objects of a concrete category |
This file defines the category of pointed objects of a concrete category. After this we will have the categories of pointed groups, pointed abelian groups, pointed groupoids, etc.
To define `Pointed.functor`, we need to add the following "pullback" construction to the category of elements.
```
@[simps obj map]
def pullback (F : D ⥤ Type w) (G : C ⥤ D) :
(G ⋙ F).Elements ⥤ F.Elements where
obj X := ⟨G.obj X.1, X.2⟩
map {X Y} f := ⟨G.map f.1, f.2⟩
```
This is called pullback since the display map of `G ⋙ F` (i.e. `π (G ⋙ F)`) is a pullback of the display map of `F`.
---
[](https://gitpod.io/from-referrer/)
|
t-category-theory
awaiting-author
|
185/0 |
Mathlib.lean,Mathlib/CategoryTheory/ConcreteCategory/Pointed.lean,Mathlib/CategoryTheory/Elements.lean |
3 |
13 |
['dagurtomas', 'github-actions', 'kim-em'] |
nobody |
386-82475 1 year ago |
408-83131 1 year ago |
7-80557 7 days |
16253 |
Shreyas4991 author:Shreyas4991 |
feat: Basics of Discrete Fair Division in Mathlib |
This PR adds the basics of discrete fair division in mathlib. We include the definitions of allocations, valuations, properties of valuations, and the following notions : Envy-Freeness (EF), Envy-Freeness upto 1 good (EF1), and envy freeness upto any good (EFX). We also include the various implications between these notions.
---
[](https://gitpod.io/from-referrer/)
|
awaiting-author
WIP
|
144/0 |
Mathlib/GameTheory/FairDivision/Discrete/Basic.lean |
1 |
9 |
['Shreyas4991', 'eric-wieser', 'github-actions'] |
nobody |
379-54524 1 year ago |
379-54524 1 year ago |
0-20853 5 hours |
14669 |
Command-Master author:Command-Master |
feat(Data/Nat/PartENat): add lemmas for PartENat |
Add some missing lemmas for `PartENat`, as well as the additive homomorphism from it to `WithTop Int`.
---
[](https://gitpod.io/from-referrer/)
|
t-data
new-contributor
awaiting-author
|
90/0 |
Mathlib/Data/Nat/PartENat.lean |
1 |
3 |
['erdOne', 'github-actions', 'urkud'] |
nobody |
376-84529 1 year ago |
376-84529 1 year ago |
0-0 0 seconds |
15121 |
Eloitor author:Eloitor |
feat: iff theorems for IsSplitEpi and IsSplitMono in opposite category |
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-category-theory
awaiting-author
|
40/0 |
Mathlib/CategoryTheory/EpiMono.lean |
1 |
3 |
['github-actions', 'joelriou', 'mattrobball'] |
nobody |
376-47474 1 year ago |
408-6733 1 year ago |
7-3203 7 days |
15895 |
madvorak author:madvorak |
feat(Computability/ContextFreeGrammar): mapping between two types of nonterminal symbols |
---
[](https://gitpod.io/from-referrer/)
|
t-computability
WIP
|
172/0 |
Mathlib/Computability/ContextFreeGrammar.lean |
1 |
43 |
['YaelDillies', 'github-actions', 'madvorak'] |
nobody |
375-64267 1 year ago |
380-11376 1 year ago |
1-43047 1 day |
12278 |
Rida-Hamadani author:Rida-Hamadani |
feat(Combinatorics/SimpleGraph): Provide iff statements for distance equal and greater than 2 |
I need these lemmas to prove that Moore graphs of girth 5 are strongly regular.
---
- [x] depends on: #11945
[](https://gitpod.io/from-referrer/)
|
t-combinatorics
awaiting-author
|
76/0 |
Mathlib/Combinatorics/SimpleGraph/Metric.lean |
1 |
2 |
['github-actions', 'leanprover-community-mathlib4-bot'] |
nobody |
375-32993 1 year ago |
375-32993 1 year ago |
1-68738 1 day |
16570 |
yuma-mizuno author:yuma-mizuno |
chore(Tactic/CategoryTheory): change `TermElabM` to `MetaM` |
Separated from #15335.
To use `Qq`, we need to modify `Qq` to support universe matching. See [Zulip](https://leanprover.zulipchat.com/#narrow/stream/144837-PR-reviews/topic/.2315335.20meta.20code.20for.20monoidal.20categories).
---
- [ ] depends on: #15335
[](https://gitpod.io/from-referrer/)
|
t-meta
WIP
|
26/15 |
Mathlib/Tactic/CategoryTheory/BicategoryCoherence.lean,Mathlib/Tactic/CategoryTheory/Coherence.lean |
2 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mergify'] |
nobody |
368-71133 1 year ago |
369-29981 1 year ago |
0-0 0 seconds |
10591 |
adri326 author:adri326 |
feat(Topology/Algebra/ConstMulAction): properties of continuous actions in Hausdorff spaces |
Defines some useful properties of `ContinuousConstSMul` group actions on Hausdorff spaces:
- `MulAction.isClosed_fixedBy`, which proves that the `fixedBy α m` set is closed
- `t2_separation_smul`, which constructs an open set `s` such that `s` and `g • s` are disjoint
- `Set.InjOn.t2_separation_smul`, the extension of `t2_separation_smul` to a set of group elements whose action is injective
---
This PR belongs my series of PR around the formalization of Rubin's theorem. `MulAction.isClosed_fixedBy` is used in several places along the proof, and the separation lemmas are primarily used in showing that `(fixedBy α g)ᶜ` and `(fixedBy α h)ᶜ` are disjoint under some intricate but fully group-theoretic condition.
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-topology
awaiting-author
label:t-algebra$ |
57/0 |
Mathlib/Topology/Algebra/ConstMulAction.lean |
1 |
9 |
['ADedecker', 'adri326', 'j-loreaux', 'jcommelin'] |
ADedecker assignee:ADedecker |
367-63125 1 year ago |
519-75863 1 year ago |
55-82183 55 days |
14704 |
Command-Master author:Command-Master |
feat(FieldTheory): define typeclass for simple extensions, and prove some properties |
Define `SimpleExtension F K`, which says that `K` is a simple field extension of `F`, and show that together with transcendentality it implies `IsFractionRing F[X] K`.
---
- [x] depends on: #14710
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-algebra
awaiting-author
WIP
label:t-algebra$ |
120/0 |
Mathlib.lean,Mathlib/FieldTheory/SimpleExtension.lean |
2 |
17 |
['Command-Master', 'acmepjz', 'github-actions', 'leanprover-community-mathlib4-bot', 'tb65536'] |
nobody |
363-4175 11 months ago |
363-4175 11 months ago |
0-0 0 seconds |
16773 |
arulandu author:arulandu |
feat(Probability/Distributions): formalize Beta distribution |
Formalize Beta distribution, using Gamma distribution as a reference. Added real-valued beta wrapper, in the manner of gamma. Thanks to @EtienneC30 for help with casting real <-> complex.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-measure-probability
awaiting-author
|
286/1 |
Mathlib.lean,Mathlib/Analysis/SpecialFunctions/Gamma/Beta.lean,Mathlib/Probability/Distributions/Beta.lean |
3 |
48 |
['EtienneC30', 'arulandu', 'github-actions', 'vihdzp'] |
arulandu assignee:arulandu |
358-7691 11 months ago |
363-4409 11 months ago |
1-21124 1 day |
10796 |
mcdoll author:mcdoll |
feat(Tactic/Positivity): non-negativity of functions |
---
This makes the `Finset.sum` and `integral_nonneg` extensions even more useful.
[](https://gitpod.io/from-referrer/)
|
t-meta
WIP
|
27/0 |
Mathlib/Tactic/Positivity/Core.lean |
1 |
1 |
['YaelDillies'] |
nobody |
328-8106 10 months ago |
570-175 1 year ago |
0-0 0 seconds |
14603 |
awueth author:awueth |
feat: degree is invariant under graph isomorphism |
---
Mathlib has the definition `SimpleGraph.Iso.mapNeighborSet` which is an equivalence between neighbor sets induced by an isomorphism. Would it be beneficial to add the same equivalence for `neighborFinset`?
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-combinatorics
WIP
|
24/0 |
Mathlib/Combinatorics/SimpleGraph/Map/Finite.lean |
1 |
11 |
['awueth', 'github-actions', 'jcommelin', 'kim-em', 'urkud'] |
nobody |
325-66476 10 months ago |
325-66476 10 months ago |
31-44440 31 days |
18630 |
tomaz1502 author:tomaz1502 |
feat(Computability.Timed): Formalization of runtime complexity of List.mergeSort |
This PR adds the formalization of the runtime complexity of the merge sort algorithm, defined in `Data/List/Sort`.
Requires: https://github.com/leanprover-community/mathlib4/pull/15451
References:
- Previous PR on mathlib3: https://github.com/leanprover-community/mathlib3/pull/14494/
- First discussion on Zulip: https://leanprover.zulipchat.com/#narrow/stream/113488-general/topic/BSc.20Final.20Project/near/220647062
- Second disussion on Zulip: https://leanprover.zulipchat.com/#narrow/stream/113488-general/topic/Formalization.20of.20Runtime.20Complexity.20of.20Sorting.20Algorithms/near/284184450
---
[](https://gitpod.io/from-referrer/)
|
t-computability
new-contributor
|
526/0 |
Mathlib.lean,Mathlib/Computability/Timed/InsertionSort.lean,Mathlib/Computability/Timed/Merge.lean,Mathlib/Computability/Timed/MergeSort.lean,Mathlib/Computability/Timed/Split.lean |
5 |
8 |
['github-actions'] |
nobody |
311-63035 10 months ago |
311-63035 10 months ago |
0-0 0 seconds |
19329 |
adomani author:adomani |
perf(CI): automatically benchmark PRs when they are opened |
This action posts the comment
```
!bench
This is an automated bench-marking that runs when a PR is opened. No need to repeat.
```
whenever a PR is *opened*. It then ignores any subsequent changes to the PR.
The automatic benching should help in catching PRs that unknowingly introduce a high performance cost, as was the case for my PR #18033.
### Note.
Running `!bench` strains the benchmarking system and it is not feasible to run it on every push. However, Sebastian, in private communication with Johan, approved of automatically benching every PR once, when it is opened.
---
[](https://gitpod.io/from-referrer/)
|
CI
WIP
|
25/0 |
.github/workflows/first_bench_is_free.yml |
1 |
12 |
['Ruben-VandeVelde', 'adomani', 'alreadydone', 'eric-wieser', 'github-actions', 'grunweg', 'jcommelin'] |
nobody |
294-12129 9 months ago |
296-1084 9 months ago |
0-1356 22 minutes |
19721 |
urkud author:urkud |
feat (WIP): formalize Moreira's version of Sard's theorem |
---
I'm in the process of migrating development to https://github.com/urkud/SardMoreira
[](https://gitpod.io/from-referrer/)
|
t-analysis |
427/1 |
Mathlib.lean,Mathlib/Analysis/Calculus/ContDiff/Defs.lean,Mathlib/Analysis/Calculus/ContDiff/FTaylorSeries.lean,Mathlib/Analysis/Calculus/ContDiff/FaaDiBruno.lean,Mathlib/Analysis/Calculus/Moreira2001.lean |
5 |
1 |
['github-actions'] |
nobody |
267-37209 8 months ago |
272-34024 8 months ago |
0-0 0 seconds |
18236 |
joelriou author:joelriou |
feat(Algebra/Category/ModuleCat/Presheaf): the endofunctor of presheaves of modules induced by an oplax natural transformation |
An endomorphism of ` ModuleCat.restrictScalarsPseudofunctor`, i.e. a "compatible" family of functors `ModuleCat A ⥤ ModuleCat A` for all (commutative) rings `A` induces a functor `PresheafOfModules R ⥤ PresheafOfModules R` for any presheaf of (commutative) rings `R`.
In #18262, this is applied to the construction of exterior powers of a presheaves of modules.
---
- [x] depends on: #18197
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-category-theory
WIP
label:t-algebra$ |
180/0 |
Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Presheaf/FunctorOfNatTrans.lean |
2 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
266-59660 8 months ago |
266-59698 8 months ago |
0-0 0 seconds |
20459 |
Ruben-VandeVelde author:Ruben-VandeVelde |
chore: fix names of roots_C_mul_X_{add,sub}_C_of_IsUnit |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
awaiting-author
label:t-algebra$ |
11/5 |
Mathlib/Algebra/Polynomial/FieldDivision.lean,Mathlib/Algebra/Polynomial/Roots.lean |
2 |
2 |
['eric-wieser', 'github-actions'] |
nobody |
247-64562 8 months ago |
247-64562 8 months ago |
4-64422 4 days |
10977 |
grunweg author:grunweg |
feat: germs of smooth functions |
Define the space of germs of smooth functions (between manifolds).
Endow it with a ring structure if the target manifold is a smooth ring (e.g., a Lie group or a field).
From the sphere eversion project, rewritten by me.
Co-authored-by: Patrick Massot
-------
Particular questions for review
- is the authorship/copyright information appropriate?
(`PatrickMassot` created the file `SmoothGerm` which I adapted; I didn't trace this far back through sphere-eversion.)
- is providing all the intermediate algebraic structures (such as, an additive subgroup) on the space of smooth germs useful in practice? (The sphere eversion project only needs a ring structure.)
- any further particular API lemmas (e.g., around coercions) which would be good to add?
---
[](https://gitpod.io/from-referrer/)
|
t-analysis
t-topology
t-differential-geometry
awaiting-author
|
150/0 |
Mathlib.lean,Mathlib/Geometry/Manifold/Algebra/SmoothGerm.lean |
2 |
33 |
['YaelDillies', 'github-actions', 'grunweg', 'jcommelin', 'kim-em', 'mcdoll'] |
fpvandoorn assignee:fpvandoorn |
247-52319 8 months ago |
381-73684 1 year ago |
144-63944 144 days |
19378 |
adamtopaz author:adamtopaz |
feat: Explanation widgets |
This adds some simple widgets, wrapped in a tactic, term and command elaborator, for displaying markdown explanations in the infoview.
---
[](https://gitpod.io/from-referrer/)
|
t-meta
awaiting-author
|
101/0 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Widget/Explain.lean |
3 |
8 |
['adamtopaz', 'eric-wieser', 'github-actions', 'joneugster', 'kmill'] |
nobody |
244-68597 8 months ago |
244-68597 8 months ago |
49-80804 49 days |
19323 |
madvorak author:madvorak |
feat: Function to Sum decomposition |
---
Discussion: https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Function.20to.20Sum.20decomposition |
t-data
WIP
|
50/0 |
Mathlib.lean,Mathlib/Data/Sum/Decompose.lean |
2 |
2 |
['github-actions', 'madvorak'] |
nobody |
242-75259 7 months ago |
252-77857 8 months ago |
43-18005 43 days |
18461 |
hannahfechtner author:hannahfechtner |
feat: left and right common multiples mixins |
add mixins for left and right common multiples. These carry the data of what factors are used to create the common multiples
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-algebra
awaiting-author
label:t-algebra$ |
78/0 |
Mathlib/Algebra/Group/Defs.lean |
1 |
13 |
['github-actions', 'hannahfechtner', 'jcommelin', 'kbuzzard', 'kim-em', 'trivial1711'] |
nobody |
236-4611 7 months ago |
236-4611 7 months ago |
69-35596 69 days |
20797 |
vbeffara author:vbeffara |
feat(Topology/Covering): CM version of eq_of_comp_eq |
Add equivalents of the lemmas `IsCoveringMap.eq_of_comp_eq` and `IsCoveringMap.const_of_comp_CM` for the case of bundled `ContinuousMap` parameters.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-topology
easy
awaiting-author
|
9/1 |
Mathlib/Topology/Covering.lean |
1 |
4 |
['github-actions', 'ocfnash', 'vbeffara'] |
nobody |
235-77776 7 months ago |
236-78729 7 months ago |
2-77310 2 days |
17589 |
joelriou author:joelriou |
feat(Algebra/ModuleCat/Presheaf): composition of pushforwards and pullbacks and compatibilites |
The composition of two pullback functors on presheaves of modules `pullback φ ⋙ pullback ψ` identifies to the pullback of the composition. We show compatibilites for these isomorphisms: they are deduced from similar identifies for pushforward (in which case they are `rfl`).
---
- [x] depends on: #17366
[](https://gitpod.io/from-referrer/)
|
t-algebraic-geometry
t-category-theory
WIP
|
166/2 |
Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Presheaf/Limits.lean,Mathlib/Algebra/Category/ModuleCat/Presheaf/Pullback.lean,Mathlib/Algebra/Category/ModuleCat/Presheaf/Pushforward.lean |
4 |
4 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
232-58442 7 months ago |
232-58461 7 months ago |
0-0 0 seconds |
21009 |
vihdzp author:vihdzp |
feat(Logic/Relation): more `TransGen` lemmas |
---
[](https://gitpod.io/from-referrer/)
|
t-logic
t-order
awaiting-author
|
13/0 |
Mathlib/Logic/Relation.lean |
1 |
2 |
['b-mehta', 'github-actions'] |
nobody |
231-73414 7 months ago |
231-73414 7 months ago |
0-39342 10 hours |
21035 |
mattrobball author:mattrobball |
draft |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
3/3 |
Mathlib/RingTheory/Kaehler/JacobiZariski.lean |
1 |
4 |
['github-actions', 'leanprover-bot', 'mattrobball'] |
nobody |
231-43954 7 months ago |
231-45793 7 months ago |
0-0 0 seconds |
15443 |
YaelDillies author:YaelDillies |
feat: The Marcinkiewicz-Zygmund inequality |
Prove the Marcinkiewicz-Zygmund inequality.
The Marcinkiewicz-Zygmund inequality states that, if `X₁, ... Xₐ ∈ L^p` are independent random
variables of mean zero valued in some inner product space, then the `L^p`-norm of `X₁ + ... + Xₐ` is
at most `Cₚ` times the `L^(p/2)`-norm of `|X₁|² + ... + |Xₐ|²`, where `Cₚ` is a constant depending on
`p` alone.
From LeanAPAP
Co-authored-by: Bhavik Mehta
---
- [x] depends on: #15832
- [x] depends on: #21033
[](https://gitpod.io/from-referrer/)
|
t-analysis
WIP
|
189/0 |
Mathlib.lean,Mathlib/Probability/MarcinkiewiczZygmund.lean |
2 |
39 |
['Parcly-Taxel', 'YaelDillies', 'b-mehta', 'github-actions', 'hrmacbeth', 'mathlib4-dependent-issues-bot', 'sgouezel'] |
nobody |
231-5356 7 months ago |
231-10420 7 months ago |
89-28229 89 days |
20466 |
MohanadAhmed author:MohanadAhmed |
feat: Sherman Morrison formula for rank 1 update of the matrix inverse |
Provides the Sherman Morrison rank 1 update of the matrix inverse https://en.wikipedia.org/wiki/Sherman%E2%80%93Morrison_formula.
---
[](https://gitpod.io/from-referrer/)
|
t-data
awaiting-author
|
37/0 |
Mathlib/Data/Matrix/Invertible.lean |
1 |
4 |
['eric-wieser', 'github-actions'] |
nobody |
228-71279 7 months ago |
228-71279 7 months ago |
23-30991 23 days |
18749 |
GabinKolly author:GabinKolly |
feat(ModelTheory): preparatory work for the existence of Fraïsse limits |
Define the map of a PartialEquiv through an embedding, and related properties.
Define embeddings and equivalences between equal structures or equal substructures, and related properties.
Add miscellaneous lemmas which will be used to prove the existence of fraisse limits.
---
This is preparation for #18876
[](https://gitpod.io/from-referrer/)
|
t-logic
awaiting-author
|
308/5 |
Mathlib/ModelTheory/Bundled.lean,Mathlib/ModelTheory/DirectLimit.lean,Mathlib/ModelTheory/FinitelyGenerated.lean,Mathlib/ModelTheory/PartialEquiv.lean,Mathlib/ModelTheory/Substructures.lean |
5 |
9 |
['GabinKolly', 'YaelDillies', 'github-actions', 'vihdzp'] |
nobody |
225-47736 7 months ago |
235-60190 7 months ago |
73-63475 73 days |
20649 |
GabinKolly author:GabinKolly |
feat(ModelTheory/Graph): prove characterization of the fraisse limit of finite simple graphs |
Prove that a countable graph with the extension property must be the Fraisse limit of finite simple graphs.
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-logic
t-combinatorics
WIP
|
175/0 |
Mathlib/ModelTheory/Graph.lean,Mathlib/ModelTheory/Substructures.lean |
2 |
1 |
['github-actions'] |
nobody |
223-43595 7 months ago |
245-41236 8 months ago |
0-0 0 seconds |
21384 |
alreadydone author:alreadydone |
experiment: make submodule quotient reducibly defeq to additive group quotient |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
1/1 |
Mathlib/LinearAlgebra/Quotient/Defs.lean |
1 |
1 |
['github-actions'] |
nobody |
221-62178 7 months ago |
221-62181 7 months ago |
0-0 0 seconds |
10660 |
eric-wieser author:eric-wieser |
feat(LinearAlgebra/CliffordAlgebra): construction from a basis |
This is adapted from https://github.com/eric-wieser/lftcm2023-clifford_algebra, which only worked for the special case of `Q = 0`.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
awaiting-author
WIP
label:t-algebra$ |
573/0 |
Mathlib.lean,Mathlib/LinearAlgebra/CliffordAlgebra/Basis.lean |
2 |
15 |
['github-actions'] |
nobody |
220-21816 7 months ago |
220-21816 7 months ago |
0-0 0 seconds |
15355 |
adomani author:adomani |
feat: MiM PR report |
---
[](https://gitpod.io/from-referrer/)
|
WIP |
153/0 |
.github/workflows/monthly_pr_report.yaml,scripts/find_labels.sh |
2 |
n/a |
['YaelDillies', 'adomani', 'github-actions'] |
nobody |
219-1738 7 months ago |
unknown |
unknown |
21495 |
alreadydone author:alreadydone |
experiment: reducible HasQuotient.quotient' |
---
[](https://gitpod.io/from-referrer/)
|
bench-after-CI
WIP
|
2/0 |
Mathlib/Algebra/Quotient.lean |
1 |
1 |
['github-actions'] |
nobody |
218-82228 7 months ago |
218-82228 7 months ago |
0-200 3 minutes |
21496 |
alreadydone author:alreadydone |
experiment: make SetLike.coe reducible |
---
[](https://gitpod.io/from-referrer/)
|
bench-after-CI
t-data
|
1/1 |
Mathlib/Data/SetLike/Basic.lean |
1 |
1 |
['github-actions'] |
nobody |
218-81997 7 months ago |
218-81997 7 months ago |
0-0 0 seconds |
21447 |
erdOne author:erdOne |
feat(AlgebraicGeometry): the split algebraic torus |
---
[](https://gitpod.io/from-referrer/)
|
t-algebraic-geometry
awaiting-author
|
419/0 |
Mathlib.lean,Mathlib/AlgebraicGeometry/Torus.lean |
2 |
4 |
['erdOne', 'github-actions', 'joelriou'] |
nobody |
217-29002 7 months ago |
217-47176 7 months ago |
2-69252 2 days |
22037 |
EtienneC30 author:EtienneC30 |
issues with Finset subtype coercion |
[Zulip discussion](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Finset.20subtype.20changes)
---
[](https://gitpod.io/from-referrer/)
|
t-data |
7/1 |
Mathlib/Data/Finset/Defs.lean,Mathlib/MeasureTheory/Constructions/Projective.lean |
2 |
1 |
['github-actions'] |
nobody |
207-625 6 months ago |
207-677 6 months ago |
0-0 0 seconds |
13442 |
dignissimus author:dignissimus |
feat: mabel tactic for multiplicative abelian groups |
Mabel tactic for multiplicative abelian groups (#10361)
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-meta
modifies-tactic-syntax
awaiting-author
help-wanted
|
439/0 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/MAbel.lean,MathlibTest/mabel.lean |
4 |
10 |
['BoltonBailey', 'dignissimus', 'github-actions', 'joneugster', 'kbuzzard'] |
joneugster assignee:joneugster |
205-43539 6 months ago |
210-25135 6 months ago |
0-16 16 seconds |
21501 |
sksgurdldi author:sksgurdldi |
feat(List): add sum_zipWith_eq_finset_sum |
### **Description:**
This PR adds the lemma `List.sum_zipWith_eq_finset_sum` to `Mathlib.Algebra.BigOperators.Group.Finset.Basic`.
#### **Statement:**
The sum of the `zipWith` operation on two lists equals the sum of applying the operation to corresponding elements of the two lists, indexed over the minimum of their lengths.
#### **Formal Statement:**
```lean
lemma sum_zipWith_eq_finset_sum [Inhabited α] [Inhabited β] [AddCommMonoid γ]
{op : α → β → γ}
(l : List α) (m : List β) :
(List.zipWith op l m).sum =
∑ x ∈ (Finset.range (Nat.min l.length m.length)), op (l[x]!) (m[x]!)
```
#### **Remarks:**
- This lemma provides a useful equivalence between `List.zipWith` and summation over a `Finset.range` indexed by `Nat.min l.length m.length`.
- It can be helpful in algebraic manipulations involving list-based summations.
#### **Dependencies:**
No additional dependencies.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-algebra
awaiting-author
label:t-algebra$ |
43/0 |
Mathlib/Algebra/BigOperators/Group/Finset/Basic.lean |
1 |
1 |
['github-actions', 'j-loreaux'] |
nobody |
205-42618 6 months ago |
205-42618 6 months ago |
13-33168 13 days |
22194 |
eric-wieser author:eric-wieser |
feat: oracle computations (alternative) |
This explores a simpler version of #20924
---
[](https://gitpod.io/from-referrer/)
|
t-computability |
698/0 |
Archive/Examples/SumOracle.lean,Mathlib.lean,Mathlib/Computability/QueryComplexity/Defs.lean,Mathlib/Computability/QueryComplexity/Sort.lean |
4 |
4 |
['eric-wieser', 'girving', 'github-actions'] |
nobody |
201-83875 6 months ago |
202-38363 6 months ago |
0-0 0 seconds |
19062 |
hannahfechtner author:hannahfechtner |
feat(Algebra/PresentedMonoid/Basic) : facts about rel |
Add in a number of useful theorems (reflexivity, closure under multiplication) and lemmas about when the PresentedMonoid.rel holds as an API for users
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
awaiting-author
label:t-algebra$ |
38/0 |
Mathlib/GroupTheory/Congruence/Defs.lean |
1 |
8 |
['github-actions', 'hannahfechtner', 'kbuzzard', 'riccardobrasca'] |
nobody |
199-80187 6 months ago |
199-80187 6 months ago |
87-64575 87 days |
22302 |
CharredLee author:CharredLee |
feat: add `CategoryTheory.Topos.Power` |
This is a continuation of #21281 with the end goal of defining topoi in Mathlib. It introduces the notion of a power object in a category with a subobject classifier, which is a special case of an internal hom.
The definition `HasPowerObjects C` contained in this PR is all that remains before `IsTopos C` can be defined.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-category-theory
awaiting-author
|
312/0 |
Mathlib.lean,Mathlib/CategoryTheory/Topos/Power.lean |
2 |
2 |
['github-actions', 'joelriou'] |
b-mehta assignee:b-mehta |
199-43814 6 months ago |
199-44941 6 months ago |
0-1528 25 minutes |
22416 |
JLimperg author:JLimperg |
chore: fix benchmark script for precompilation |
The benchmarking script used to fail when precompilation was enabled anywhere in the dependency graph.
---
Fix courtesy of @Kha.
[](https://gitpod.io/from-referrer/)
|
|
2/0 |
scripts/bench/fake-root/lib/lean/libleanshared.so,scripts/bench/run |
2 |
1 |
['github-actions'] |
nobody |
196-39869 6 months ago |
196-39932 6 months ago |
0-0 0 seconds |
22389 |
adomani author:adomani |
feat: the variableVariable linter |
The motivation comes from [this Zulip discussion](https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/style.20proposal.3A.20avoid.20.60variable.20.7BX.7D.20.2E.2E.2E.20variable.20.28X.29.60).
Summarising, updating a variable binder for a single declaration can be confusing.
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-linter
WIP
|
167/0 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter.lean,Mathlib/Tactic/Linter/VariableVariable.lean,variableDeclarationVariable_replacements.py |
5 |
1 |
['github-actions'] |
nobody |
194-67336 6 months ago |
197-2092 6 months ago |
0-0 0 seconds |
22497 |
adomani author:adomani |
test: decl diff in lean |
Testing branch for #22464.
---
[](https://gitpod.io/from-referrer/)
|
test-ci
CI
WIP
|
161/0 |
.github/workflows/PR_summary_lean.yml,Mathlib.lean,Mathlib/Test.lean,scripts/README.md,scripts/declarations_diff.lean,scripts/declarations_diff_lean_shell_glue.sh |
6 |
7 |
['github-actions', 'mergify'] |
nobody |
192-66914 6 months ago |
193-78613 6 months ago |
0-0 0 seconds |
20636 |
eric-wieser author:eric-wieser |
feat: multiplication of intervals in rings |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
awaiting-author
label:t-algebra$ |
36/1 |
Mathlib/Algebra/Order/Interval/Basic.lean |
1 |
16 |
['Timeroot', 'YaelDillies', 'eric-wieser', 'github-actions'] |
nobody |
192-55535 6 months ago |
228-59312 7 months ago |
17-17852 17 days |
22648 |
adomani author:adomani |
test: lean implementation decl diff quandle |
---
[](https://gitpod.io/from-referrer/)
|
|
210/1 |
.github/workflows/PR_summary_lean.yml,Mathlib/Algebra/Quandle.lean,scripts/README.md,scripts/declarations_diff.lean,scripts/declarations_diff_lean_shell_glue.sh |
5 |
4 |
['adomani', 'eric-wieser', 'github-actions'] |
nobody |
189-11294 6 months ago |
190-66980 6 months ago |
0-0 0 seconds |
22784 |
grunweg author:grunweg |
feat: add Diffeomorph.sumSumSumComm |
This matches `{Equiv,Homeomorph.sumSumSumComm}`, and is needed to prove that addition in the cobordism group is commutatives. From my bordism theory project.
---
- depends on #22783 (easy pre-requisites)
The current proof is not complete yet, and feels very painful. I'm not yet sure what's the best way to write this.
[](https://gitpod.io/from-referrer/)
|
t-differential-geometry
WIP
|
50/0 |
Mathlib/Geometry/Manifold/Diffeomorph.lean |
1 |
1 |
['github-actions'] |
nobody |
186-51367 6 months ago |
186-74111 6 months ago |
0-0 0 seconds |
22846 |
mattrobball author:mattrobball |
test |
|
t-analysis |
2/0 |
Mathlib/Analysis/Normed/Module/Basic.lean |
1 |
4 |
['github-actions', 'leanprover-bot', 'mattrobball'] |
nobody |
185-55875 6 months ago |
185-57815 6 months ago |
0-0 0 seconds |
22159 |
shetzl author:shetzl |
feat: add definition of pushdown automata |
Add the definition of pushdown automata and their two acceptance conditions: acceptance based on empty stack and acceptance based on final state.
Co-authored-by: Tobias Leichtfried
---
[](https://gitpod.io/from-referrer/)
|
t-computability
new-contributor
awaiting-author
|
70/0 |
Mathlib.lean,Mathlib/Computability/PDA.lean |
2 |
34 |
['YaelDillies', 'github-actions', 'madvorak', 'shetzl'] |
nobody |
180-4961 5 months ago |
180-4961 5 months ago |
20-81771 20 days |
23042 |
joneugster author:joneugster |
feat(CategoryTheory/Enriched/Limits): add HasConicalLimitsOfSize.shrink |
---
Note: I've marked this "WIP" because I'm not yet sure when this will be needed and I'd probably put the PR on the queue once I've created some follow-up needing it.
[](https://gitpod.io/from-referrer/)
|
infinity-cosmos
t-category-theory
WIP
|
22/1 |
Mathlib/CategoryTheory/Enriched/Limits/HasConicalLimits.lean |
1 |
1 |
['github-actions'] |
nobody |
179-3073 5 months ago |
179-3228 5 months ago |
0-1 1 second |
17587 |
kmill author:kmill |
feat: Sym2-as-Finset theory |
---
[](https://gitpod.io/from-referrer/)
|
t-data
new-contributor
|
105/3 |
Mathlib/Combinatorics/SimpleGraph/Basic.lean,Mathlib/Combinatorics/SimpleGraph/Finite.lean,Mathlib/Data/Sym/Sym2.lean,Mathlib/RingTheory/Polynomial/Vieta.lean |
4 |
10 |
['FordUniver', 'YaelDillies', 'github-actions', 'kmill'] |
nobody |
178-15486 5 months ago |
178-50966 5 months ago |
0-0 0 seconds |
16239 |
Rida-Hamadani author:Rida-Hamadani |
feat(Geometry/Manifold): orientable manifolds |
This module defines orientable manifolds. [This](https://leanprover.zulipchat.com/#narrow/stream/217875-Is-there-code-for-X.3F/topic/Orientable.20Surface) Zulip topic is related.
---
[](https://gitpod.io/from-referrer/)
|
t-differential-geometry
awaiting-author
|
376/6 |
Mathlib.lean,Mathlib/Geometry/Manifold/Instances/Real.lean,Mathlib/Geometry/Manifold/Orientable.lean |
3 |
39 |
['Rida-Hamadani', 'github-actions', 'grunweg', 'ocfnash'] |
nobody |
176-38133 5 months ago |
195-76855 6 months ago |
5-70530 5 days |
23142 |
joneugster author:joneugster |
feat(CategoryTheory/Enriched/Limits): add API for HasConicalLimit |
---
[](https://gitpod.io/from-referrer/)
|
infinity-cosmos
t-category-theory
awaiting-author
|
52/9 |
Mathlib/CategoryTheory/Enriched/Limits/HasConicalLimits.lean |
1 |
2 |
['github-actions', 'joelriou'] |
nobody |
176-6219 5 months ago |
176-6219 5 months ago |
0-68906 19 hours |
23285 |
AntoineChambert-Loir author:AntoineChambert-Loir |
refactor: directed systems in terms of functors |
This is a WIP aiming to refactor the work on directed systems using the category theory library.
But there are universes nightmares.
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebra
t-category-theory
WIP
label:t-algebra$ |
111/45 |
Mathlib/Order/DirectedInverseSystem.lean |
1 |
1 |
['github-actions'] |
nobody |
172-43010 5 months ago |
172-43016 5 months ago |
0-24 24 seconds |
21829 |
Whysoserioushah author:Whysoserioushah |
feat(LinearAlgebra/TensorProduct/HomTensor): Add TensorProduct of Hom-modules |
Co-authored-by: Andrew Yang
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
awaiting-author
label:t-algebra$ |
174/0 |
Mathlib.lean,Mathlib/LinearAlgebra/TensorProduct/HomTensor.lean |
2 |
26 |
['Whysoserioushah', 'YaelDillies', 'erdOne', 'github-actions', 'kbuzzard'] |
nobody |
163-85633 5 months ago |
165-5753 5 months ago |
46-53384 46 days |
22861 |
eric-wieser author:eric-wieser |
feat: add the trace of a bilinear form |
Following the steps at [#Is there code for X? > Laplacian @ 💬](https://leanprover.zulipchat.com/#narrow/channel/217875-Is-there-code-for-X.3F/topic/Laplacian/near/450834505).
---
[](https://gitpod.io/from-referrer/)
Some questions:
* Does this generalize to multilinear maps?
* Is there an `RCLike` generalization?
* Does this generalize to `BilinMap` instead of just `BilinForm`?
Perhaps the approach in [#mathlib4 > Stating Schrodinger's equation @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Stating.20Schrodinger's.20equation/near/500409890) of using `ContinuousLinearMap.adjoint'` is better.
|
t-algebra
awaiting-author
label:t-algebra$ |
100/0 |
Mathlib.lean,Mathlib/LinearAlgebra/BilinearForm/Trace.lean |
2 |
3 |
['github-actions', 'jcommelin'] |
nobody |
161-75472 5 months ago |
161-75472 5 months ago |
23-44995 23 days |
22888 |
plp127 author:plp127 |
perf: replace `Lean.Expr.swapBVars` with a better? implementation |
Replaces `Lean.Expr.swapBVars` with a version that traverses the expression.
---
[](https://gitpod.io/from-referrer/)
|
t-meta
awaiting-author
|
14/12 |
Mathlib/Tactic/FunProp/ToBatteries.lean |
1 |
23 |
['eric-wieser', 'github-actions', 'joneugster', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'plp127'] |
eric-wieser and joneugster assignee:eric-wieser assignee:joneugster |
159-1318 5 months ago |
159-74017 5 months ago |
4-80306 4 days |
23772 |
SEU-Prime author:SEU-Prime |
Create Amice.lean |
i built amice equiv
[](https://gitpod.io/from-referrer/)
|
t-number-theory
WIP
|
283/0 |
Mathlib/NumberTheory/Padics/Amice.lean |
1 |
2 |
['grunweg'] |
nobody |
158-74166 5 months ago |
158-74166 5 months ago |
0-8688 2 hours |
21903 |
yhtq author:yhtq |
feat: add from/toList between `FreeSemigroup` and `List` with relative theorems |
Add from/toList between `FreeSemigroup` and `List` with relative theorems, as well as an incidental definition of lexicographic order on `FreeSemigroup`.
---
[](https://gitpod.io/from-referrer/)
|
large-import
new-contributor
t-algebra
awaiting-CI
label:t-algebra$ |
169/0 |
Mathlib/Algebra/Free.lean |
1 |
11 |
['YaelDillies', 'github-actions'] |
nobody |
158-20287 5 months ago |
158-20287 5 months ago |
51-9403 51 days |
22657 |
Xmask19 author:Xmask19 |
feat: a graph is maximally acyclic iff it is a tree |
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-combinatorics
|
86/0 |
Mathlib/Combinatorics/SimpleGraph/Acyclic.lean |
1 |
6 |
['Rida-Hamadani', 'b-mehta', 'github-actions', 'grunweg'] |
b-mehta assignee:b-mehta |
157-72344 5 months ago |
157-72365 5 months ago |
179-63035 179 days |
21342 |
YaelDillies author:YaelDillies |
refactor(Normed/Group/Quotient): generalise to non-abelian groups |
The goal is to apply this to the free group.
---
- [x] depends on: #21341
[](https://gitpod.io/from-referrer/)
|
t-analysis
WIP
|
25/12 |
Mathlib/Topology/Algebra/ConstMulAction.lean,Mathlib/Topology/Algebra/Group/Quotient.lean |
2 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
155-11529 5 months ago |
155-11548 5 months ago |
0-352 5 minutes |
24000 |
YaelDillies author:YaelDillies |
feat: correspondence between Hopf algebras and affine group schemes |
Construct `Spec` as a functor from `R`-Hopf algebras to group schemes over `Spec R`, show it is full and faithful and has affine group schemes as essential image.
From Toric, FLT
Co-authored-by: Andrew Yang
Co-authored-by: Michał Mrugała
Co-authored-by: Christian Merten
---
[](https://gitpod.io/from-referrer/)
|
toric
FLT
t-algebraic-geometry
WIP
|
127/0 |
Mathlib/AlgebraicGeometry/GroupScheme/HopfAffine.lean |
1 |
3 |
['YaelDillies', 'github-actions', 'kbuzzard'] |
nobody |
152-42926 4 months ago |
152-80878 4 months ago |
0-1 1 second |
21270 |
GabinKolly author:GabinKolly |
feat(ModelTheory/Bundled): first-order embeddings and equivalences from equalities |
Add first-order embeddings and equivalences from equalities between bundled structures.
---
Add two definitions to get embeddings and equivalences from equalities between bundled structures, and simple properties.
This is some preparatory work for #18876
[](https://gitpod.io/from-referrer/)
|
large-import
t-logic
awaiting-author
|
102/0 |
Mathlib/ModelTheory/Bundled.lean |
1 |
26 |
['GabinKolly', 'Vierkantor', 'YaelDillies', 'github-actions'] |
nobody |
152-12899 4 months ago |
152-12899 4 months ago |
50-58472 50 days |
24086 |
mattrobball author:mattrobball |
perf(Normed.Field.Basic): change parent order for `Semifield` and `Field` and reduce priority `toComm(Semi)Ring` |
Passing through the projection `toComm(Semi)Ring` should not be preferred.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
8/2 |
Mathlib/Algebra/Field/Defs.lean |
1 |
4 |
['github-actions', 'leanprover-bot', 'mattrobball'] |
nobody |
150-65936 4 months ago |
150-70736 4 months ago |
0-0 0 seconds |
13038 |
adomani author:adomani |
feat: Mathlib weekly reports |
This PR introduces a weekly cron job that computes a "global" report on the evolution of Mathlib in the previous week.
It consists of
* a CI workflow with a cron job that runs at minight on Sunday (`.github/workflows/mathlib_stats.yaml`);
* a Lean file extracting a categorized list of "all" the declarations in Mathlib (`scripts/count_decls.lean`);
* a bash file computing Git-diff-related information and collating the data from the Lean file (`scripts/mathlib_stats.sh`);
* a convenience CI workflow that is triggered on adding the `test-ci` label and results in posting on the PR and on Zulip the report (`.github/workflows/mathlib_stats_label.yaml`).
The second CI workflow is intended to be removed just before/right after the PR is ready to merge.
[Zulip discussion](https://leanprover.zulipchat.com/#narrow/stream/113488-general)
[Thread for the reports](https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/Mathlib.20weekly.20change.20report)
---
[](https://gitpod.io/from-referrer/)
|
CI
t-meta
awaiting-author
|
338/0 |
.github/workflows/mathlib_stats.yaml,.github/workflows/mathlib_stats_label.yaml,scripts/count_decls.lean,scripts/mathlib_stats.sh |
4 |
10 |
['adomani', 'github-actions', 'grunweg', 'kim-em', 'kmill'] |
nobody |
150-46890 4 months ago |
424-64770 1 year ago |
57-4216 57 days |
24129 |
urkud author:urkud |
feat: symmetry of Gateaux derivatives |
---
[](https://gitpod.io/from-referrer/)
|
t-analysis |
190/1 |
Mathlib.lean,Mathlib/Analysis/Calculus/LineDeriv/Basic.lean,Mathlib/Analysis/Calculus/LineDeriv/Symmetric.lean |
3 |
1 |
['github-actions'] |
nobody |
149-14117 4 months ago |
149-14117 4 months ago |
0-0 0 seconds |
19613 |
madvorak author:madvorak |
refactor(Combinatorics/Optimization/ValuedCSP): make only valid `FractionalOperation` possible |
Originally `FractionalOperation` was any multiset (possible empty).
Then `FractionalOperation.IsValid` said it was nonempty.
Instead, I would like to make it nonempty by definition.
As a result, empty/invalid fractional operation couldn't be declared at all.
---
[](https://gitpod.io/from-referrer/)
|
t-combinatorics |
14/17 |
Mathlib/Combinatorics/Optimization/ValuedCSP.lean |
1 |
1 |
['github-actions'] |
nobody |
148-50334 4 months ago |
277-71907 9 months ago |
287-59545 287 days |
23600 |
mattrobball author:mattrobball |
perf(Quiver.Basic): make `IsThin` a `class` |
It seems problematic that `Quiver.IsThin` is an `abbrev` for (essentially) `Subsingleton`. We turn it in a one-field class.
---
[](https://gitpod.io/from-referrer/)
|
delegated |
27/21 |
Mathlib/CategoryTheory/Bicategory/Coherence.lean,Mathlib/CategoryTheory/Category/Preorder.lean,Mathlib/CategoryTheory/Generator/Basic.lean,Mathlib/CategoryTheory/Groupoid/Basic.lean,Mathlib/CategoryTheory/Limits/Shapes/WidePullbacks.lean,Mathlib/CategoryTheory/Limits/SmallComplete.lean,Mathlib/CategoryTheory/Monoidal/Free/Coherence.lean,Mathlib/CategoryTheory/Skeletal.lean,Mathlib/CategoryTheory/Subobject/MonoOver.lean,Mathlib/CategoryTheory/Thin.lean,Mathlib/Combinatorics/Quiver/Basic.lean |
11 |
16 |
['b-mehta', 'github-actions', 'leanprover-bot', 'mathlib-bors', 'mattrobball'] |
nobody |
147-67469 4 months ago |
162-66273 5 months ago |
0-5717 1 hour |
24219 |
Paul-Lez author:Paul-Lez |
feat: linear independence of the tensor product of two linearly independent families |
This is still WIP (the proofs are a little too long, and some lemmas need to be moved to other files!)
From Toric
---
[](https://gitpod.io/from-referrer/)
|
toric
t-algebra
WIP
label:t-algebra$ |
193/0 |
Mathlib/LinearAlgebra/LinearIndependent/Tprod.lean |
1 |
1 |
['github-actions'] |
nobody |
143-69167 4 months ago |
143-69167 4 months ago |
0-2221 37 minutes |
13740 |
YaelDillies author:YaelDillies |
feat: More robust ae notation |
Make sure that, when `μ : FiniteMeasure Ω`, `f =ᵐ[μ] g` elaborates to `f =ᵐ[↑μ] g` instead of complaining about `OuterMeasureClass (FiniteMeasure Ω) (Set Ω) ℝ≥0∞` not existing.
[Zulip](https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/ae.20of.20a.20finite.20measure)
---
[](https://gitpod.io/from-referrer/)
|
t-measure-probability
awaiting-CI
t-meta
|
56/2 |
Mathlib/MeasureTheory/Measure/MeasureSpaceDef.lean,Mathlib/MeasureTheory/OuterMeasure/AE.lean,Mathlib/MeasureTheory/OuterMeasure/BorelCantelli.lean |
3 |
16 |
['YaelDillies', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'urkud'] |
nobody |
143-7239 4 months ago |
143-7254 4 months ago |
0-0 0 seconds |
24161 |
urkud author:urkud |
feat(Analysis/Calculus/Schwarzian): new file |
---
[](https://gitpod.io/from-referrer/)
|
t-analysis |
190/3 |
Mathlib.lean,Mathlib/Analysis/Calculus/Deriv/ZPow.lean,Mathlib/Analysis/Calculus/Schwarzian/Basic.lean |
3 |
2 |
['github-actions', 'leanprover-community-bot-assistant'] |
nobody |
142-80493 4 months ago |
142-80511 4 months ago |
0-0 0 seconds |
20652 |
jjaassoonn author:jjaassoonn |
feat: categorical description of center of a ring |
We show the isomorphism between `Z(R)` and `End(1 Mod-R)`
---
- [x] depends on:#20721
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-category-theory
awaiting-author
label:t-algebra$ |
212/21 |
Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/ChangeOfRings.lean,Mathlib/Algebra/Category/Ring/Center.lean,Mathlib/CategoryTheory/Conj.lean,Mathlib/CategoryTheory/Endomorphism.lean,Mathlib/CategoryTheory/Preadditive/AdditiveFunctor.lean,Mathlib/CategoryTheory/Preadditive/Basic.lean |
7 |
41 |
['alreadydone', 'github-actions', 'jcommelin', 'jjaassoonn', 'kbuzzard', 'qawbecrdtey'] |
nobody |
142-36605 4 months ago |
200-2286 6 months ago |
20-7596 20 days |
21616 |
peabrainiac author:peabrainiac |
feat(Topology): concatenating countably many paths |
Adds `Path.countableConcat`, the concatenation of a sequence of paths leading up to some point `x`.
---
- [x] depends on: #21591
- [x] depends on: #21607
This work is a prerequisite to #20248, where it is used to show that the topology of first-countable locally path-connected spaces is coinduced by all the paths in that space.
[](https://gitpod.io/from-referrer/)
|
t-topology
awaiting-author
|
229/0 |
Mathlib.lean,Mathlib/Topology/Path/CountableConcat.lean |
2 |
30 |
['YaelDillies', 'github-actions', 'kim-em', 'mathlib4-dependent-issues-bot', 'peabrainiac'] |
YaelDillies assignee:YaelDillies |
142-2528 4 months ago |
146-10462 4 months ago |
56-56728 56 days |
18210 |
vihdzp author:vihdzp |
feat(Order/Hom/Basic): `WithBot (Fin n) ≃o Fin (n + 1)` |
---
[](https://gitpod.io/from-referrer/)
|
t-order
awaiting-author
|
16/0 |
Mathlib/Order/Hom/Basic.lean |
1 |
8 |
['Command-Master', 'Ruben-VandeVelde', 'github-actions', 'urkud', 'vihdzp'] |
nobody |
141-35236 4 months ago |
312-39314 10 months ago |
10-77913 10 days |
23585 |
plp127 author:plp127 |
feat: `Filter.atMax` and `Filter.atMin` |
Adds `atMax` and `atMin`, filters. Making an analogy, `atMax` : `atTop` :: `IsMax` : `IsTop`.
---
[](https://gitpod.io/from-referrer/)
|
t-order
WIP
|
148/0 |
Mathlib.lean,Mathlib/Order/Filter/AtMaxMin.lean |
2 |
4 |
['github-actions', 'plp127', 'urkud'] |
nobody |
141-26045 4 months ago |
164-703 5 months ago |
0-0 0 seconds |
12032 |
mcdoll author:mcdoll |
feat: Delta distribution as a limit |
---
- [x] depends on: #11496
[](https://gitpod.io/from-referrer/)
|
t-analysis
WIP
|
51/0 |
Mathlib/Analysis/Distribution/DiracDelta.lean |
1 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
138-40840 4 months ago |
unknown |
unknown |
24157 |
urkud author:urkud |
feat(Convex/LinearIsometry): new file |
---
- [x] depends on: #24392
[](https://gitpod.io/from-referrer/)
|
t-analysis
awaiting-author
|
75/0 |
Mathlib.lean,Mathlib/Analysis/Convex/LinearIsometry.lean |
2 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'sgouezel'] |
nobody |
136-7773 4 months ago |
136-7773 4 months ago |
10-23076 10 days |
18861 |
YaelDillies author:YaelDillies |
refactor: make `Set.mem_graphOn` defeq |
The definition as an image is cute but not very useful. Also unsimp `graphOn_univ` since the RHS contains `f` more times than the LHS does.
---
Later, I would like to introduce `Set.graph` to have a `Set` version with good defeqs of `LinearMap.graph` and alike
[](https://gitpod.io/from-referrer/)
|
t-data
awaiting-author
|
72/18 |
Mathlib/Data/Set/Function.lean,Mathlib/Data/Set/Operations.lean,Mathlib/Data/Set/Prod.lean,Mathlib/MeasureTheory/Covering/Besicovitch.lean |
4 |
4 |
['YaelDillies', 'b-mehta', 'github-actions'] |
nobody |
133-15513 4 months ago |
173-55222 5 months ago |
2-24624 2 days |
23503 |
apnelson1 author:apnelson1 |
feat(Topology/Instances/ENat): ENat and tsum |
We give API for the interactions between `tsum` and `ENat`. The type is especially nice, because every function is summable, and there are simplifying lemmas like the statement that a sum is infinite iff either some term is infinite, or the support is infinite.
This provides one of the missing pieces for working painlessly with discrete objects, 'propositional' finiteness and cardinality. For instance, one can sum a function `f : a -> ENat` over an arbitrary set with the term `∑' a : s, 1`, and it will be provable that `∑' a : s, 1 = s.encard` and `(support f).encard ≤ ∑' a, f a` without ever having to split into finite/infinite cases.
As is pointed out in the module docstring for `Data.ENat`, there are strong analogies between `ENat` and `ENNReal`, and the API runs parallel to the API for `tsum`/`ENNReal`. One could call it 'duplication', but I have yet to find a common generalization of the two that saves work, or a third example of a natural type with these same properties.
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-topology
WIP
|
205/2 |
Mathlib/Data/ENat/Basic.lean,Mathlib/Data/Set/Card.lean,Mathlib/Topology/Instances/ENat.lean |
3 |
2 |
['eric-wieser', 'github-actions'] |
nobody |
133-11394 4 months ago |
133-11394 4 months ago |
14-6036 14 days |
22809 |
b-reinke author:b-reinke |
feat: Category algebras and path algebras |
This PR defines the category algebra of a linear category and path algebras of quivers.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-algebra
t-category-theory
WIP
label:t-algebra$ |
218/0 |
Mathlib/Algebra/Ring/Assoc.lean,Mathlib/CategoryTheory/Linear/CategoryAlgebra.lean,Mathlib/Combinatorics/Quiver/PathAlgebra.lean,Mathlib/Data/DFinsupp/BigOperators.lean |
4 |
2 |
['b-reinke', 'github-actions'] |
nobody |
133-11358 4 months ago |
133-11358 4 months ago |
0-0 0 seconds |
19797 |
eric-wieser author:eric-wieser |
refactor: use Qq in the nlinarith preprocessor |
This also provides the machinery needed to Qq-ify linarith itself.
This is still doing far more `synthInstanceQ`/`isDefEq`(`Q`) than should be needed, but at least drops the `mkAppM`s.
Currently, this takes a different approach to the one used by `NormNum.Result`:
* `NormNum.Result` deliberately avoids adding any `Expr` parameters to types, as this makes defeq problem at compile-time hard
* This PR allows the Expr parameters, but adds casting helpers to easily transport along defeq(Q)s. A few `unsafeIntro`s are left, which correspond to either a Qq bug, or a flaw in the idea behind this approach.
I don't know if this pattern is an improvement.
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-meta
|
260/28 |
Mathlib/Data/Ineq.lean,Mathlib/Tactic/Linarith/Datatypes.lean,Mathlib/Tactic/Linarith/Oracle/SimplexAlgorithm.lean,Mathlib/Tactic/Linarith/Preprocessing.lean,Mathlib/Util/Qq.lean |
5 |
8 |
['eric-wieser', 'github-actions', 'leanprover-bot'] |
nobody |
133-11080 4 months ago |
133-11080 4 months ago |
0-0 0 seconds |
14348 |
eric-wieser author:eric-wieser |
perf: disable the `unusedVariables` linter for speed |
I doubt we want to merge this, but it shaves two minutes of the lint time.
---
[](https://gitpod.io/from-referrer/)
|
performance-hack |
1/0 |
lakefile.lean |
1 |
3 |
['eric-wieser', 'github-actions', 'leanprover-bot'] |
nobody |
133-10388 4 months ago |
133-10388 4 months ago |
0-0 0 seconds |
24574 |
JovanGerb author:JovanGerb |
chore(Order/Notation): check for pp options in `delabSup` |
The sup/inf delaborator shouldn't run when the user sets `pp.explicit true` or `pp.notation false`.
This PR also removes my "-- TODO(Jovan): remove"
edit: apparently, the fix in core wasn't fully successful. There still isn't support for adding/storing the localInstance inside `PPContext` or `MessageDataContext`. So we need that, or we need to extract the local instances anyways.
---
[](https://gitpod.io/from-referrer/)
|
t-order |
8/12 |
Mathlib/Order/Notation.lean |
1 |
1 |
['github-actions'] |
nobody |
132-32068 4 months ago |
132-52842 4 months ago |
132-52886 132 days |
22488 |
smmercuri author:smmercuri |
fix: lower priority for `UniformSpace.Completion.instSMul` |
Following the introduction of the `WithVal` type synonym in #22055 the following instance takes a long time to synthesise in FLT, and times out in the default heartbeats
```lean
import Mathlib
namespace IsDedekindDomain.HeightOneSpectrum
variable (A K : Type*) [CommRing A] [Field K] [Algebra A K] [IsFractionRing A K]
[IsDedekindDomain A] (v : HeightOneSpectrum A)
#synth SMul (v.adicCompletionIntegers K) (v.adicCompletion K)
```
The issue is that `UniformSpace.Completion.instSMul (v.adicCompletionIntegers K) (v.adicCompletion K)` now fires during the start of instance search (because we now have `UniformSpace (WithVal (v.valuation K))` whereas previously this would be `UniformSpace K`, which was not automatic), and this takes a long time to fail (leading to ~1400 entries in the trace). The first few lines of the new trace is
```lean
[Meta.synthInstance] [5.512418] ✅️ SMul (↥(adicCompletionIntegers K v)) (adicCompletion K v) ▼
[] [0.000118] new goal SMul (↥(adicCompletionIntegers K v)) (adicCompletion K v) ▶
[] [0.000537] ✅️ apply UniformSpace.Completion.instSMul to SMul (↥(adicCompletionIntegers K v)) (adicCompletion K v) ▶
[] [0.004411] ✅️ apply @WithVal.instSMul to SMul (↥(adicCompletionIntegers K v)) (WithVal (valuation K v)) ▶
[] [0.000765] ❌️ apply @GradedMonoid.GradeZero.smul to SMul (↥(adicCompletionIntegers K v)) K ▶
[] [0.000378] ✅️ apply @Algebra.toSMul to SMul (↥(adicCompletionIntegers K v)) K ▶
...
[] 1339 more entries... ▶
```
Lowering the priority of `UniformSpace.Completion.instSMul` fixes this particular issue, leading to a trace that matches that seen prior to the introduction of `WithVal`:
```lean
[Meta.synthInstance] [0.016405] ✅️ SMul (↥(adicCompletionIntegers K v)) (adicCompletion K v) ▼
[] [0.000119] new goal SMul (↥(adicCompletionIntegers K v)) (adicCompletion K v) ▶
[] [0.000491] ❌️ apply @GradedMonoid.GradeZero.smul to SMul (↥(adicCompletionIntegers K v)) (adicCompletion K v) ▶
[] [0.000403] ✅️ apply @Algebra.toSMul to SMul (↥(adicCompletionIntegers K v)) (adicCompletion K v) ▶
[] [0.000134] ❌️ apply inst✝⁴ to Algebra (↥(adicCompletionIntegers K v)) (adicCompletion K v) ▶
[] [0.000093] ❌️ apply inst✝⁵ to Algebra (↥(adicCompletionIntegers K v)) (adicCompletion K v) ▶
[] [0.000077] ❌️ apply inst✝⁷ to Algebra (↥(adicCompletionIntegers K v)) (adicCompletion K v) ▶
[] [0.000082] ❌️ apply inst✝⁹ to Algebra (↥(adicCompletionIntegers K v)) (adicCompletion K v) ▶
[] [0.000075] ❌️ apply inst✝¹² to Algebra (↥(adicCompletionIntegers K v)) (adicCompletion K v) ▶
[] [0.000220] ❌️ apply Algebra.id to Algebra (↥(adicCompletionIntegers K v)) (adicCompletion K v) ▶
[] [0.001015] ✅️ apply @ValuationSubring.instAlgebraSubtypeMem to Algebra (↥(adicCompletionIntegers K v))
(adicCompletion K v) ▶
[resume] [0.000038] propagating Algebra (↥(adicCompletionIntegers K v))
(adicCompletion K
v) to subgoal Algebra (↥(adicCompletionIntegers K v))
(adicCompletion K v) of SMul (↥(adicCompletionIntegers K v)) (adicCompletion K v) ▶
[check] [0.013358] ✅️ Algebra.toSMul
[] result Algebra.toSMul
```
---
[](https://gitpod.io/from-referrer/)
|
FLT
t-topology
awaiting-author
|
1/1 |
Mathlib/Topology/Algebra/UniformMulAction.lean |
1 |
10 |
['github-actions', 'leanprover-bot', 'smmercuri', 'urkud'] |
nobody |
131-80572 4 months ago |
138-22724 4 months ago |
55-70108 55 days |
15161 |
adomani author:adomani |
feat(Linter): flag `intros x y` which can be replaced by `intro x y` |
---
[](https://gitpod.io/from-referrer/)
|
t-linter
WIP
|
78/1 |
Mathlib/Tactic/Linter/Lint.lean,test/Lint.lean |
2 |
4 |
['adomani', 'github-actions', 'grunweg'] |
nobody |
131-51640 4 months ago |
131-86254 4 months ago |
0-0 0 seconds |
15649 |
TpmKranz author:TpmKranz |
feat(Computability): introduce Generalised NFA as bridge to Regular Expression |
Lays the groundwork for a proof of equivalence of NFA and RE, w.r.t. described language. Actual connection to NFA comes later, after the groundwork for the opposite direction has been laid.
Second chunk of #12648
---
- [x] depends on: #15647 [Data.FinEnum.Option unchanged since then]
[](https://gitpod.io/from-referrer/)
|
awaiting-zulip
t-computability
new-contributor
awaiting-author
|
298/0 |
Mathlib.lean,Mathlib/Computability/GNFA.lean,Mathlib/Computability/Language.lean,Mathlib/Computability/RegularExpressions.lean,docs/references.bib |
5 |
6 |
['github-actions', 'mathlib4-dependent-issues-bot', 'meithecatte', 'trivial1711'] |
nobody |
130-44077 4 months ago |
130-44086 4 months ago |
23-54870 23 days |
20648 |
anthonyde author:anthonyde |
feat: formalize regular expression -> εNFA |
The file `Computability/RegularExpressionsToEpsilonNFA.lean` contains a formal definition of Thompson's method for constructing an `εNFA` from a `RegularExpression` and a proof of its correctness.
---
- [x] depends on: #20644
- [x] depends on: #20645
[](https://gitpod.io/from-referrer/)
|
awaiting-zulip
t-computability
new-contributor
|
490/0 |
Mathlib.lean,Mathlib/Computability/RegularExpressionsToEpsilonNFA.lean,docs/references.bib |
3 |
5 |
['github-actions', 'mathlib4-dependent-issues-bot', 'meithecatte', 'qawbecrdtey'] |
nobody |
130-43388 4 months ago |
130-44023 4 months ago |
75-77754 75 days |
23220 |
mattrobball author:mattrobball |
refactor(Module.LinearMap.Defs): make `SemilinearMapClass` extend `AddMonoidHomClass` |
Currently `SemilinearMapClass` extends `AddHomClass`. As both `SemilinearMapClass.toAddHomClass` and `AddMonoidHomClass.toAddHomClass` are projections, they have the same priority. With `SemilinearMapClass` declared later, it wins causing expensive failed searches in the algebraic hierarchy before `AddMonoidHomClass.toAddHomClass` is found.
The current instance `SemilinearMapClass.toAddMonoidHomClass` has lower priority so we may need to downgrade the priority of the projection also.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
awaiting-author
label:t-algebra$ |
6/10 |
Mathlib/Algebra/Module/LinearMap/Defs.lean |
1 |
9 |
['eric-wieser', 'github-actions', 'leanprover-bot', 'mattrobball'] |
nobody |
129-45523 4 months ago |
129-45523 4 months ago |
45-6308 45 days |
24665 |
Komyyy author:Komyyy |
feat(Mathlib/Topology/Metrizable/Uniformity): every uniform space is generated by a family of pseudometrics |
---
[](https://gitpod.io/from-referrer/)
|
t-topology
WIP
|
54/0 |
Mathlib/Topology/Metrizable/Uniformity.lean |
1 |
1 |
['github-actions'] |
nobody |
128-54297 4 months ago |
128-54297 4 months ago |
0-1 1 second |
23213 |
mattrobball author:mattrobball |
chore(RingTheory.Derivation): add a `LinearMapClass` instance |
Often we want `simp` to call `map_zero` or `map_add` for a `Derivation`. To find the `ZeroHomClass` or `AddHomClass` instance necessary it starts to climb up the type class hierarchy including looking for a `LinearMapClass` instance which didn't exist. Consequently, sythesis would look in a lot of crazy places trying to summon ring structures on the module or on derivations itself. Here we add the missing `LinearMapClass` instance so that `simp` is more efficient.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
delegated
label:t-algebra$ |
5/3 |
Mathlib/RingTheory/Derivation/Basic.lean |
1 |
8 |
['github-actions', 'j-loreaux', 'leanprover-bot', 'mathlib-bors', 'mattrobball'] |
nobody |
127-44735 4 months ago |
127-44735 4 months ago |
47-39026 47 days |
23214 |
mattrobball author:mattrobball |
perf(Module.LinearMap.Defs): deprioritize projections to parents for `SemilinearMapClass` |
Trying to figure out if a given type has a `SemilinearMapClass` instance when all we want is an `AddHomClass` or a `MulActionSemiHomClass` can be quite expensive since there are multiple ways to crawl the algebraic hierarchy to generate `LinearMapClass` instances. If these fail, then they fail slowly. We deprioritize the projections from `SemilinearMapClass` to `AddHomClass` and `MulActionSemiHomClass` to make this one of the last choices.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
delegated
label:t-algebra$ |
6/0 |
Mathlib/Algebra/Module/LinearMap/Defs.lean |
1 |
6 |
['github-actions', 'j-loreaux', 'leanprover-bot', 'mathlib-bors', 'mattrobball'] |
nobody |
127-44501 4 months ago |
127-44501 4 months ago |
47-32152 47 days |
24155 |
eric-wieser author:eric-wieser |
feat: add a "rw_proc" for fin vectors |
This seems a little nicer than an elaborator, since it means I can use the default elaboration rules to handle my first few variables.
Ideally there would be something like
```lean
rw_procQ {A : Type u} {B : A -> Type v} (a : A) (b : B a) : b = ?rhs => do
/-- Context:
u v : Level
A : Q(Type u)
B : Q($A -> Type v)
a : Q($A)
b : Q($B $a)
rhs : Q($B $a) -- metavariable to assign
|- MetaM Q($b = ?rhs)
-/
```
or
```lean
rw_proc {A : Type u} {B : A -> Type v} (a : A) (b : B a) : b = ?rhs => do
/-- Context:
u v : Level
A B a b : Expr
rhs : MVarId
|- MetaM Expr
-/
```
which would generate the code I wrote here
---
[](https://gitpod.io/from-referrer/)
|
t-data
RFC
t-meta
awaiting-author
|
27/2 |
Mathlib/Data/Fin/Tuple/Reflection.lean |
1 |
2 |
['github-actions', 'urkud'] |
nobody |
127-41878 4 months ago |
127-41878 4 months ago |
20-83091 20 days |
22314 |
shetzl author:shetzl |
feat: add leftmost derivations for context-free grammars |
Leftmost derivations are often easier to reason about than arbitrary derivations. This PR adds leftmost variants of Rewrites, Produces and Derives to the existing definition of context-free grammars and proves that a string of terminals can be derived iff it can be leftmost derived.
Co-authored-by: Tobias Leichtfried
---
[](https://gitpod.io/from-referrer/)
|
t-computability
new-contributor
awaiting-author
|
383/0 |
Mathlib.lean,Mathlib/Computability/LeftmostDerivation.lean |
2 |
54 |
['YaelDillies', 'github-actions', 'madvorak', 'shetzl'] |
YaelDillies assignee:YaelDillies |
127-2352 4 months ago |
127-2352 4 months ago |
72-3718 72 days |
21276 |
GabinKolly author:GabinKolly |
feat(ModelTheory/Substructures): define equivalences between equal substructures |
Define first-order equivalences between equal substructures, and prove related properties.
---
This is some preparatory work for #18876
[](https://gitpod.io/from-referrer/)
|
t-logic
awaiting-author
|
62/0 |
Mathlib/ModelTheory/Substructures.lean |
1 |
19 |
['GabinKolly', 'YaelDillies', 'fpvandoorn', 'github-actions', 'grunweg'] |
nobody |
126-64072 4 months ago |
126-64072 4 months ago |
46-55730 46 days |
23137 |
grunweg author:grunweg |
chore(Topology): some more fun_prop tagging |
---
[](https://gitpod.io/from-referrer/)
|
t-topology
delegated
|
8/4 |
Mathlib/Dynamics/Flow.lean,Mathlib/Topology/Algebra/Monoid.lean |
2 |
10 |
['github-actions', 'grunweg', 'j-loreaux', 'mathlib-bors'] |
nobody |
126-46950 4 months ago |
126-46950 4 months ago |
34-32727 34 days |
24532 |
robertmaxton42 author:robertmaxton42 |
feat(LinearAlgebra/FreeProduct): fill out the `FreeProduct.asPowers` namespace |
* Replicate the existing API for `LinearAlgebra.FreeProduct` under `FreeProduct.asPowers`, for convenience when working primarily with the power algebra representation
* Adds convenience lemmas for using the corresponding quotient relation `rel'` (used in the above).
---
- [x] depends on: #24531
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
122/5 |
Mathlib/LinearAlgebra/FreeProduct/Basic.lean |
1 |
25 |
['YaelDillies', 'adomani', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'robertmaxton42'] |
nobody |
125-8032 4 months ago |
125-8084 4 months ago |
125-56382 125 days |
24008 |
meithecatte author:meithecatte |
chore(EpsilonNFA): replace manual lemmas with @[simps] |
---
[](https://gitpod.io/from-referrer/)
|
t-computability
new-contributor
awaiting-author
|
2/24 |
Mathlib/Computability/EpsilonNFA.lean |
1 |
2 |
['YaelDillies', 'github-actions', 'urkud'] |
nobody |
125-3216 4 months ago |
125-3216 4 months ago |
27-52316 27 days |
24744 |
Timeroot author:Timeroot |
Post's lattice |
Draft PR for now so I can get CI checks. Eventually want to prove Post's Lattice
---
[](https://gitpod.io/from-referrer/)
|
WIP |
758/0 |
Mathlib.lean,Mathlib/Algebra/Clone/Basic.lean,Mathlib/Algebra/Clone/Defs.lean,Mathlib/Algebra/Clone/Instances.lean,Mathlib/Algebra/Clone/PostLattice.lean,Mathlib/Data/Fin/Basic.lean |
6 |
1 |
['github-actions'] |
nobody |
123-9685 4 months ago |
123-9685 4 months ago |
0-0 0 seconds |
24618 |
b-mehta author:b-mehta |
feat(Analysis): add Schur inequality and variants |
Add Schur inequality and some of its common variants.
TODO:
- [x] add reference to source: https://www.cip.ifi.lmu.de/~grinberg/VornicuS.pdf
- [ ] add other generalisations
- [ ] move some of the lemmas elsewhere
---
[](https://gitpod.io/from-referrer/)
|
t-analysis
WIP
|
145/0 |
Mathlib/Analysis/Convex/Schur.lean |
1 |
16 |
['b-mehta', 'eric-wieser', 'github-actions'] |
nobody |
121-77149 3 months ago |
130-57087 4 months ago |
0-2 2 seconds |
24957 |
eric-wieser author:eric-wieser |
feat: use ` binderNameHint` in sum_congr |
Zulip thread: [#new members > Choosing dummy variable inside summation @ 💬](https://leanprover.zulipchat.com/#narrow/channel/113489-new-members/topic/Choosing.20dummy.20variable.20inside.20summation/near/518492888)
Co-authored-by: Joachim Breitner
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
23/16 |
Mathlib/Algebra/BigOperators/Expect.lean,Mathlib/Algebra/BigOperators/Group/Finset/Basic.lean,Mathlib/Analysis/BoxIntegral/Partition/Basic.lean,Mathlib/Data/Finset/Fold.lean,Mathlib/Data/Finset/Lattice/Fold.lean,Mathlib/Data/List/OfFn.lean,Mathlib/Data/Multiset/Count.lean,Mathlib/Data/Multiset/Filter.lean,Mathlib/Data/Multiset/MapFold.lean,Mathlib/Data/Option/Basic.lean,Mathlib/Data/Set/Image.lean,Mathlib/Data/Sym/Basic.lean,Mathlib/Data/Sym/Sym2.lean |
13 |
1 |
['github-actions'] |
nobody |
119-76293 3 months ago |
119-77743 3 months ago |
119-77796 119 days |
5919 |
MithicSpirit author:MithicSpirit |
feat: implement orthogonality for AffineSubspace |
Define `AffineSubspace.orthogonal` and `AffineSubspace.IsOrtho`, as well as develop an API emulating that of `Submodule.orthogonal` and `Submodule.IsOrtho`, respectively. Additionally, provide some relevant lemmas exclusive to affine subspaces, which are mostly to do with the relationship between orthogonality and `AffineSubspace.Parallel`.
Closes #5539
---
Still WIP as I need to add more docstrings as well as notations for the new definitions.
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-analysis
WIP
help-wanted
|
287/0 |
Mathlib.lean,Mathlib/Analysis/InnerProductSpace/AffineSubspace.lean |
2 |
6 |
['MithicSpirit', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant'] |
MithicSpirit assignee:MithicSpirit |
118-59762 3 months ago |
118-59780 3 months ago |
0-0 0 seconds |
10235 |
urkud author:urkud |
feat: add `Decidable`, `Fintype`, `Encodable` linters |
This PR ports the `decidableClassical`, `fintypeFinite` and `encodableCountable` linters from mathlib3: all three are environment linters which flag declarations that have a hypothesis `[Decidable p]` etc., but do not use the underlying assumption in this type. Restructuring the code can make the statement more general.
The implementation is in fact quite general, and can easily adapt to include further types. PRs #17518 and #17519 are two examples of further such linters.
---
Please don't fix the failures related to `HasFDerivWithinAt.pi`. Finiteness assumptions in these lemmas will be completely removed during porting to TVS.
[](https://gitpod.io/from-referrer/) |
awaiting-bench
large-import
t-linter
t-meta
awaiting-author
|
123/4 |
Mathlib.lean,Mathlib/Computability/Halting.lean,Mathlib/Computability/TuringMachine.lean,Mathlib/Data/Fintype/Quotient.lean,Mathlib/Logic/Basic.lean,Mathlib/Logic/Encodable/Basic.lean,Mathlib/NumberTheory/JacobiSum/Basic.lean,Mathlib/Order/Heyting/Regular.lean,Mathlib/Tactic.lean,Mathlib/Tactic/GeneralizeProofs.lean,Mathlib/Tactic/Linter/UnusedAssumptionInType.lean |
11 |
n/a |
['Command-Master', 'github-actions', 'grunweg', 'kmill', 'leanprover-bot', 'urkud'] |
nobody |
118-58459 3 months ago |
unknown |
unknown |
22539 |
joelriou author:joelriou |
feat(Algebra/Homology): construction of left resolutions |
Given a fully faithful functor `ι : C ⥤ A` to an abelian category, we introduce a structure `Abelian.LeftResolutions ι` which gives a functor `F : A ⥤ C` and a natural epimorphism `π.app X : ι.obj (F.obj X) ⟶ X` for all `X : A`. This is used in order to construct a resolution functor `LeftResolutions.chainComplexFunctor : A ⥤ ChainComplex C ℕ`.
This shall be used in order to derive the tensor product of modules and sheaves of modules.
---
[](https://gitpod.io/from-referrer/)
|
t-category-theory
WIP
|
271/19 |
Mathlib.lean,Mathlib/Algebra/Homology/HomologicalComplex.lean,Mathlib/Algebra/Homology/LeftResolutions/Basic.lean,Mathlib/CategoryTheory/Limits/Shapes/Kernels.lean |
4 |
1 |
['github-actions'] |
nobody |
117-81290 3 months ago |
133-70108 4 months ago |
59-17063 59 days |
21624 |
sinhp author:sinhp |
feat(CategoryTheory): The (closed) monoidal structure on the product category of families of (closed) monoidal categories |
Given a family of closed monoidal categories, we show that the product of these categories
is a closed monoidal category with the pointwise monoidal structure.
---
[](https://gitpod.io/from-referrer/)
|
t-category-theory
awaiting-author
|
144/0 |
Mathlib.lean,Mathlib/CategoryTheory/Pi/Basic.lean,Mathlib/CategoryTheory/Pi/Monoidal.lean,Mathlib/CategoryTheory/Pi/MonoidalClosed.lean |
4 |
19 |
['TwoFX', 'YaelDillies', 'b-mehta', 'github-actions', 'jcommelin', 'sinhp'] |
nobody |
116-11589 3 months ago |
116-11589 3 months ago |
54-54882 54 days |
11155 |
smorel394 author:smorel394 |
feat(LinearAlgebra/Multilinear/DirectSum, LinearAlgebra/DirectSum/{PiTensorProduct,Finsupp}): interaction between `MultilinearMap` and `DirectSum`, and between `PiTensorProduct` and `DirectSum` |
This does three things:
* `MultilinearMap.fromDirectSumEquiv` (in `LinearAlgebra/MultilinearMap/DirectSum.lean`) calculates `MultilinearMap`s on a family of `DirectSum`s. More precisely, if `ι` is a `Fintype`, if `κ i` is a family of types indexed by `ι` and we have a `R`-module `M i j` for every `i : ι` and `j : κ i`, this is the linear equivalence between `Π p : (i : ι) → κ i, MultilinearMap R (fun i ↦ M i (p i)) M'` and `MultilinearMap R (fun i ↦ ⨁ j : κ i, M i j) M'`.
* `PiTensorProduct.directSum` (in `LinearAlgebra/DirectSum/PiTensorProduct.lean`): the distributivity property of a `PiTensorProduct` with respect to `DirectSum`s in all its arguments.
* `finsuppPiTensorProduct` (in `LinearAlgebra/DirectSum/Finsupp.lean`): If `ι` is a `Fintype`, `κ i` is a family of types indexed by `ι` and `M i` is a family of `R`-modules indexed by `ι`, then the tensor product of the family `κ i →₀ M i` is linearly equivalent to `∏ i, κ i →₀ ⨂[R] i, M i`.
- [x] depends on: #11152
- [x] depends on: #11196
- [x] depends on: #17881
- [x] depends on: #17932
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
please-adopt
label:t-algebra$ |
322/0 |
Mathlib.lean,Mathlib/LinearAlgebra/DFinsupp/PiTensorProduct.lean,Mathlib/LinearAlgebra/DirectSum/Finsupp.lean,Mathlib/LinearAlgebra/DirectSum/PiTensorProduct.lean,Mathlib/LinearAlgebra/Multilinear/DFinsupp.lean,Mathlib/LinearAlgebra/Multilinear/DirectSum.lean |
6 |
32 |
['Ruben-VandeVelde', 'eric-wieser', 'github-actions', 'mathlib4-dependent-issues-bot', 'smorel394'] |
nobody |
112-35350 3 months ago |
112-37555 3 months ago |
6-23591 6 days |
19456 |
AntoineChambert-Loir author:AntoineChambert-Loir |
feat(Data/Finsupp/MonomialOrder/DegRevLex): homogeneous reverse lexicographic order |
Definition of the homogeneous reverse lexicographic order
---
- [x] depends on: #19453
- [x] depends on: #19455
[](https://gitpod.io/from-referrer/)
|
t-data
t-order
t-algebraic-geometry
WIP
|
362/0 |
Mathlib.lean,Mathlib/Data/Finsupp/MonomialOrder/DegLex.lean,Mathlib/Data/Finsupp/MonomialOrder/DegRevLex.lean |
3 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
111-61407 3 months ago |
111-61407 3 months ago |
0-1720 28 minutes |
24690 |
ScottCarnahan author:ScottCarnahan |
feat (Data.Prod): Reverse lexicographic order |
This PR implements the type synonym RevLex as a one-field structure, defines an order on products, and proves an order isomorphism with the Lex product with factors switched.
---
[](https://gitpod.io/from-referrer/)
|
t-order
WIP
|
141/0 |
Mathlib.lean,Mathlib/Data/Prod/RevLex.lean |
2 |
4 |
['ScottCarnahan', 'YaelDillies', 'github-actions'] |
YaelDillies assignee:YaelDillies |
108-16452 3 months ago |
108-28145 3 months ago |
19-33859 19 days |
23426 |
idontgetoutmuch author:idontgetoutmuch |
G-Bundle and examples |
---
[](https://gitpod.io/from-referrer/)
|
t-differential-geometry
awaiting-author
|
691/0 |
Mathlib/Topology/FiberBundle/Instances/GBundleDefs.lean,Mathlib/Topology/FiberBundle/Instances/Mobius.lean,Mathlib/Topology/FiberBundle/Instances/MobiusAsGBundle.lean |
3 |
4 |
['eric-wieser', 'idontgetoutmuch'] |
nobody |
107-85704 3 months ago |
119-11622 3 months ago |
0-0 0 seconds |
22919 |
plp127 author:plp127 |
feat(Data/Fintype/Pi): Make `Fintype` instance for `RelHom`s computable |
Makes the `Fintype` instance for rel homs computable.
See this [Zulip](https://leanprover.zulipchat.com/#narrow/channel/113489-new-members/topic/Classical.20vs.20constructive.20logic.20in.20computation/near/496220816) message.
---
- [x] depends on: #24748
[](https://gitpod.io/from-referrer/)
|
t-data
awaiting-author
|
178/44 |
Mathlib/Combinatorics/SimpleGraph/Basic.lean,Mathlib/Combinatorics/SimpleGraph/Coloring.lean,Mathlib/Combinatorics/SimpleGraph/Maps.lean,Mathlib/Data/Fintype/CardEmbedding.lean,Mathlib/Data/Fintype/Pi.lean |
5 |
29 |
['IvanRenison', 'b-mehta', 'eric-wieser', 'fpvandoorn', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'plp127'] |
b-mehta assignee:b-mehta |
107-24193 3 months ago |
107-24193 3 months ago |
73-73341 73 days |
25170 |
eric-wieser author:eric-wieser |
refactor: make basis computable |
I claim that in the long run, `Basis.repr` should be a `DFinsupp` not `Finsupp`, so that it is computable.
To make this change incrementally, we can store a `DFinsupp` internally today, and keep `repr` and `ofRepr` working with finsupp.
This at least would allow building a large basis object, and then using `repr'` to compute with it.
The cost of this intermediate state is a loss of many defeqs.
---
- [ ] depends on: #25166
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebra
label:t-algebra$ |
66/21 |
Mathlib/LinearAlgebra/Basis/Basic.lean,Mathlib/LinearAlgebra/Basis/Defs.lean,Mathlib/LinearAlgebra/FreeModule/Basic.lean |
3 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
106-39845 3 months ago |
107-4843 3 months ago |
0-0 0 seconds |
24065 |
kim-em author:kim-em |
chore: script to give topological sort of modules |
This script is not useful by itself: it just gives a topological sort of Mathlib's import graph. But I've several times found it useful when I want to modify many files systematically with minimal rebuilding: just work backwards through the list.
|
awaiting-author |
96/0 |
scripts/README.md,scripts/topological_sort.py |
2 |
5 |
['github-actions', 'jcommelin', 'kim-em'] |
jcommelin assignee:jcommelin |
103-15620 3 months ago |
103-15620 3 months ago |
48-7769 48 days |
20238 |
maemre author:maemre |
feat(Computability/DFA): Closure of regular languages under some set operations |
This shows that regular languages are closed under complement and intersection by constructing DFAs for them.
---
Closure under all other operations will be proved when someone adds the proof for DFA<->regular expression equivalence, so they are not part of this PR.
[](https://gitpod.io/from-referrer/)
|
awaiting-zulip
t-computability
new-contributor
awaiting-author
|
159/0 |
Mathlib/Computability/DFA.lean,Mathlib/Computability/Language.lean |
2 |
59 |
['EtienneC30', 'YaelDillies', 'github-actions', 'maemre', 'meithecatte', 'urkud'] |
EtienneC30 assignee:EtienneC30 |
101-9848 3 months ago |
130-43987 4 months ago |
48-67492 48 days |
25429 |
Paul-Lez author:Paul-Lez |
feat(Analysis/PDE/Quasilinear/Defs): Add definitions about quasilinear first order PDEs |
This PR introduces some basic definitions related to first order quasilinear PDEs.
In a subsequent PR (I'm currently cleaning up the code), these will be used to state and prove some results about how solutions to quasilinear PDEs vary along characteristic curves.
---
[](https://gitpod.io/from-referrer/)
|
t-analysis |
141/0 |
Mathlib.lean,Mathlib/Analysis/PDE/Quasilinear/Defs.lean |
2 |
1 |
['github-actions'] |
nobody |
100-77733 3 months ago |
100-85903 3 months ago |
0-0 0 seconds |
25473 |
adomani author:adomani |
feat(CI): check that Mathlib files have lean or md extension |
Twice recently there have been files with an "intended" `.lean` extension in `Mathlib/`:
* #24942, ending in `;lean`;
* #25457, ending in `.Lean`.
`mk_all` does not add these files to `Mathlib.lean`, since they do not end in `.lean` and this later causes problems.
This CI step checks that all files in `Mathlib/` end with `.lean` or `.md`.
See #25474 for a test where the new step [correctly fails](https://github.com/leanprover-community/mathlib4/actions/runs/15464097783/job/43532018379?pr=25474).
---
[](https://gitpod.io/from-referrer/)
|
CI
delegated
|
10/0 |
.github/workflows/lint_and_suggest_pr.yml |
1 |
10 |
['adomani', 'bryangingechen', 'github-actions', 'grunweg', 'mathlib-bors'] |
nobody |
99-78524 3 months ago |
99-79414 3 months ago |
0-11212 3 hours |
24441 |
MrSumato author:MrSumato |
feat(Data/List): add Lyndon-Schutzenberger theorem on list commutativity |
Add Lyndon-Schutzenberger theorem on list commutativity. Included definition for List.repeatSelf that returns list repeated n times.
---
This is my first mathlib PR, so any comments are highly appreciated.
[](https://gitpod.io/from-referrer/)
|
t-data
new-contributor
awaiting-author
|
129/1 |
Mathlib.lean,Mathlib/Data/List/Commutativity.lean,Mathlib/Data/List/Defs.lean,Mathlib/Data/List/Lemmas.lean |
4 |
35 |
['MrSumato', 'github-actions', 'grunweg', 'plp127'] |
grunweg assignee:grunweg |
98-78025 3 months ago |
98-78025 3 months ago |
29-59355 29 days |
23240 |
urkud author:urkud |
feat(Topology/Maps): `IsOpenMap` and `ClusterPt` |
---
[](https://gitpod.io/from-referrer/)
|
t-topology
delegated
|
17/4 |
Mathlib/Topology/Maps/Basic.lean |
1 |
8 |
['eric-wieser', 'github-actions', 'grunweg', 'mathlib-bors', 'urkud'] |
nobody |
98-73446 3 months ago |
173-42427 5 months ago |
0-12104 3 hours |
23929 |
meithecatte author:meithecatte |
feat(Computability/NFA): improve bound on pumping lemma |
---
- [x] depends on: #25321
[](https://gitpod.io/from-referrer/)
|
awaiting-zulip
t-computability
new-contributor
|
101/10 |
Mathlib/Computability/EpsilonNFA.lean,Mathlib/Computability/NFA.lean |
2 |
41 |
['YaelDillies', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'meithecatte'] |
nobody |
97-53639 3 months ago |
97-53640 3 months ago |
34-10595 34 days |
25579 |
JovanGerb author:JovanGerb |
feat(Order/Notation): only allow ⊔/⊓ for non-linear orders |
⊔/⊓ is the same as max/min. The difference is that it is meant to be used if and only if there is no linear order. This PR implements a check for one of the two directions.
---
[](https://gitpod.io/from-referrer/)
|
t-order |
33/7 |
Mathlib/Order/Notation.lean |
1 |
1 |
['github-actions'] |
nobody |
97-347 3 months ago |
97-29283 3 months ago |
0-0 0 seconds |
25035 |
ScottCarnahan author:ScottCarnahan |
feat (Algebra/Module/Equiv/Defs): Linear equivalence between linear hom and semilinear hom. |
Given a ring homomorphism `σ₂ : R →+* R₂`, an `R`-module `M`, and a module `M₂` for both `R` and `R₂` satisfying `SMulCommClass R R₂ M₂` and `(σ₂ r) • x = r • x`, we produce an `R₂`-linear equivalence between `M →ₗ[R] M₂` and `M →ₛₗ[σ₂] M₂`.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
WIP
label:t-algebra$ |
21/0 |
Mathlib/Algebra/Module/Equiv/Defs.lean |
1 |
1 |
['github-actions'] |
nobody |
96-13056 3 months ago |
96-13056 3 months ago |
20-7584 20 days |
25034 |
ScottCarnahan author:ScottCarnahan |
feat (Algebra/Module/Equiv/Basic): Restriction of scalars from a semilinear equivalence to a linear equivalence. |
If `M` and `M₂` are both `R`-modules and modules for `S` and `S₂`, respectively, then for any ring isomorphism `e` between `S` and `S₂` and any `e`-semilinear equivalence between `M` and `M₂` that respects the `R`-action, we obtain an `R`-linear equivalence between `M` and `M₂`.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
WIP
label:t-algebra$ |
28/0 |
Mathlib/Algebra/Module/Equiv/Basic.lean |
1 |
1 |
['github-actions'] |
nobody |
96-13031 3 months ago |
96-13031 3 months ago |
20-11468 20 days |
24540 |
robertmaxton42 author:robertmaxton42 |
feat(Quiv): add the empty, vertex, point, interval, and walking quivers |
Add:
* The empty quiver
* The vertex quiver (one vertex, and no edges) and the point quiver (one vertex, one self-edge)
* The interval quiver (two vertices with an edge between them)
* The walking quiver (vertices `0` and `1` with two edges both `0 -> 1`. Functors from the walking quiver to `Type` define quivers, by interpreting `F.obj 0` as the type of vertices, `F.obj 1` as the type of edges, using one of the two edges to label the source of every edge and using the other to label the target.)
- [x] depends on: #24538
---
[](https://gitpod.io/from-referrer/)
|
t-category-theory
awaiting-author
|
370/0 |
Mathlib.lean,Mathlib/CategoryTheory/Category/Quiv/Shapes.lean,Mathlib/CategoryTheory/Category/Quiv/WalkingQuiver.lean,Mathlib/Logic/Small/Defs.lean |
4 |
13 |
['github-actions', 'joelriou', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'robertmaxton42', 'robin-carlier'] |
nobody |
94-78454 3 months ago |
98-42467 3 months ago |
0-80193 22 hours |
22790 |
mhk119 author:mhk119 |
feat: Extend `taylor_mean_remainder_lagrange` to `x < x_0` |
The `taylor_mean_remainder_lagrange` theorem has the assumption that $x_0 < x$. In many applications, we need $x < x_0$ and one cannot use the current version to obtain this (see [zulip](https://leanprover.zulipchat.com/#narrow/channel/116395-maths/topic/Taylor's.20theorem)). This PR introduces a set of theorems that push negations through Taylor expansions so that one can extend `taylor_mean_remainder_lagrange` to the case when $x < x_0$. These theorems should also be useful elsewhere since they are quite general. |
new-contributor
t-analysis
awaiting-author
|
111/1 |
Mathlib/Analysis/Calculus/Deriv/Basic.lean,Mathlib/Analysis/Calculus/IteratedDeriv/Lemmas.lean,Mathlib/Analysis/Calculus/Taylor.lean |
3 |
12 |
['Paul-Lez', 'github-actions', 'grunweg', 'mhk119'] |
nobody |
94-38144 3 months ago |
155-79840 5 months ago |
30-77130 30 days |
21344 |
kbuzzard author:kbuzzard |
chore: attempt to avoid diamond in OreLocalization |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
please-adopt
label:t-algebra$ |
16/5 |
Mathlib/RingTheory/OreLocalization/Basic.lean |
1 |
6 |
['erdOne', 'github-actions', 'kbuzzard'] |
nobody |
94-35722 3 months ago |
94-37813 3 months ago |
53-20069 53 days |
25683 |
eric-wieser author:eric-wieser |
feat: Enumeration of NonemptyInterval |
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-data
|
52/4 |
Mathlib/Data/Sym/Sym2/Fin.lean,Mathlib/Data/Sym/Sym2/Order.lean |
2 |
1 |
['github-actions'] |
nobody |
94-34748 3 months ago |
94-34748 3 months ago |
0-0 0 seconds |
25746 |
robin-carlier author:robin-carlier |
feat(Tactic/CategoryTheory): `Cancelable` boilerplate for the `rotate_isos` WIP tactic |
This PR adds some boilerplate that will be used in a forthcoming PR implementing a `rotate_isos` tactic that aims to provide easy ways of moving one or more morphisms that can be inferred to be isomorphisms (not necessarily through the `IsIso typeclass, but also directly by recognizing them as e.g components of natural isomorphisms, or functor application to such morphisms).
The boilerplate in this PR abstracts the notion of a cancelable expression for a morphism in a composition of (iso)morphisms in a category, and records a global reference to a list of "cancelable factories", _i.e_ functions that try to recognize term in an expression as a "cancelable" morphism, and provides helper to register such functions.
---
First part of a series of 3 PRs contributing the `rotate_isos` tactic to mathlib. Second part will actually implement the tactic, and provide a test suite. Please read the description of the second PR (#24454) to get more details.
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #24452.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/24452* |
t-category-theory
t-meta
awaiting-author
|
162/0 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/CategoryTheory/RotateIsos/Cancelable.lean,scripts/noshake.json |
4 |
1 |
['github-actions'] |
nobody |
93-9805 3 months ago |
93-9834 3 months ago |
0-0 0 seconds |
25585 |
Paul-Lez author:Paul-Lez |
feat(Tactic/Linters/DeprecatedSimpLemma): lint for deprecated simp lemmas |
The deprecated simp lemma linter flags declarations that have both the `deprecated` and `simp` attributes.
See Zulip discussion: [#mathlib4 > Help with Mathlib.Order.Interval.Finset.Defs @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Help.20with.20Mathlib.2EOrder.2EInterval.2EFinset.2EDefs/near/505994843)
---
[](https://gitpod.io/from-referrer/)
|
t-linter
awaiting-author
|
105/0 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter/DeprecatedSimpLemma.lean,MathlibTest/DeprecatedSimpLemmaTest.lean |
4 |
7 |
['adomani', 'github-actions', 'grunweg'] |
nobody |
93-5918 3 months ago |
96-48135 3 months ago |
0-34675 9 hours |
25802 |
dagurtomas author:dagurtomas |
feat(AlgebraicTopology): anodyne morphisms of simplicial sets |
---
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #20201.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/20201* |
t-topology
WIP
|
148/0 |
Mathlib.lean,Mathlib/AlgebraicTopology/Anodyne.lean,Mathlib/AlgebraicTopology/KanFibration.lean,Mathlib/CategoryTheory/MorphismProperty/WeakSaturation.lean |
4 |
1 |
['github-actions'] |
nobody |
92-85006 3 months ago |
92-85023 3 months ago |
0-2 2 seconds |
25835 |
erdOne author:erdOne |
WIP: Weierstrass elliptic functions |
---
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #21662.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/21662* |
t-analysis
WIP
|
1461/0 |
Mathlib/Analysis/Elliptic/Basic.lean |
1 |
1 |
['github-actions'] |
nobody |
92-4783 3 months ago |
92-4825 3 months ago |
0-33 33 seconds |
25838 |
Bergschaf author:Bergschaf |
feat(Order/Atoms): Finsets are Atomistic |
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-order
|
31/0 |
Mathlib/Order/Atoms.lean |
1 |
1 |
['github-actions'] |
nobody |
91-84465 2 months ago |
91-84465 2 months ago |
0-0 0 seconds |
25765 |
JovanGerb author:JovanGerb |
feat(gcongr): lemma for rewriting inside divisibility |
TODO: add test to show that we can rewrite using `a ≡ b [ZMOD n]` inside `n ∣ 2 * a + 1`.
edit: it's not yet entirely clear if this is the right thing to do.
---
[](https://gitpod.io/from-referrer/)
|
t-data
delegated
|
5/0 |
Mathlib/Data/Int/ModEq.lean |
1 |
3 |
['fpvandoorn', 'github-actions', 'mathlib-bors'] |
nobody |
91-36961 2 months ago |
91-72499 2 months ago |
1-19951 1 day |
25871 |
eric-wieser author:eric-wieser |
refactor: generalize rank lemmas to semirings |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
18/8 |
Mathlib/LinearAlgebra/Dimension/Finite.lean |
1 |
1 |
['github-actions'] |
nobody |
90-64422 2 months ago |
90-64448 2 months ago |
0-0 0 seconds |
25911 |
BoltonBailey author:BoltonBailey |
make `a / b` simp normal form |
This PR continues the work from #25631.
Original PR: https://github.com/leanprover-community/mathlib4/pull/25631 |
t-algebra label:t-algebra$ |
11/1 |
Mathlib/Algebra/Group/Defs.lean |
1 |
2 |
['BoltonBailey', 'github-actions'] |
nobody |
89-70212 2 months ago |
89-70215 2 months ago |
0-0 0 seconds |
25918 |
BoltonBailey author:BoltonBailey |
feat: one time pad string diagram |
This PR continues the work from #10655.
Original PR: https://github.com/leanprover-community/mathlib4/pull/10655 |
|
159/0 |
MathlibTest/StringDiagram.lean |
1 |
2 |
['BoltonBailey', 'github-actions'] |
nobody |
89-68356 2 months ago |
89-68444 2 months ago |
0-0 0 seconds |
25990 |
Multramate author:Multramate |
chore(NumberTheory/EllipticDivisibilitySequence): rename definitions |
This PR continues the work from #25132.
Original PR: https://github.com/leanprover-community/mathlib4/pull/25132 |
t-number-theory |
265/45 |
Mathlib/NumberTheory/EllipticDivisibilitySequence.lean |
1 |
2 |
['Multramate', 'github-actions'] |
nobody |
88-44261 2 months ago |
88-44261 2 months ago |
0-0 0 seconds |
25987 |
Multramate author:Multramate |
refactor(AlgebraicGeometry/EllipticCurve/Affine/*): some minor changes |
This PR continues the work from #24571.
Original PR: https://github.com/leanprover-community/mathlib4/pull/24571 |
t-algebraic-geometry |
0/12 |
Mathlib.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Group.lean |
2 |
n/a |
['Multramate', 'github-actions', 'grunweg'] |
nobody |
88-4422 2 months ago |
unknown |
unknown |
25921 |
BoltonBailey author:BoltonBailey |
feat: scripts to analyze overlap between namespaces |
This PR continues the work from #11385.
Original PR: https://github.com/leanprover-community/mathlib4/pull/11385 |
migrated-from-branch
t-meta
WIP
|
86/0 |
scripts/RecordNamespaces.lean,scripts/namespace-overlap.py |
2 |
1 |
['github-actions'] |
nobody |
87-56223 2 months ago |
87-56223 2 months ago |
2-11832 2 days |
26085 |
grunweg author:grunweg |
feat: disjoint unions distribute with products of manifolds |
This PR continues the work from #22611.
Original PR: https://github.com/leanprover-community/mathlib4/pull/22611 |
t-differential-geometry
please-adopt
WIP
|
75/6 |
Mathlib/Geometry/Manifold/Diffeomorph.lean,Mathlib/Geometry/Manifold/LocalDiffeomorph.lean |
2 |
2 |
['github-actions', 'grunweg'] |
nobody |
86-78281 2 months ago |
86-78283 2 months ago |
0-74 1 minute |
25971 |
joelriou author:joelriou |
feat(CategoryTheory): pseudofunctors to Cat |
This PR adds convenience lemmas for pseudofunctors to `Cat`, mostly using the `to_app` attribute. The simp set for the `to_app` attribute is extended in order to take into account that in `Cat`, associators and unitors induce identities.
---
This PR continues the work from #24384.
Original PR: https://github.com/leanprover-community/mathlib4/pull/24384 |
t-category-theory
awaiting-author
|
142/8 |
Mathlib.lean,Mathlib/CategoryTheory/Bicategory/Functor/Cat.lean,Mathlib/CategoryTheory/Bicategory/Functor/Strict.lean,Mathlib/Tactic/CategoryTheory/ToApp.lean,MathlibTest/CategoryTheory/ToApp.lean |
5 |
6 |
['callesonne', 'chrisflav', 'github-actions', 'joelriou'] |
nobody |
86-72381 2 months ago |
86-74906 2 months ago |
0-7170 1 hour |
26174 |
grunweg author:grunweg |
feat: split continuous linear maps |
We define split linear maps and prove their basic properties.
Manually migrated from #23186.
---
There are two sorries left. One is `ClosedComplemented.prod`; the other relates to the composition of split maps. Help with both is welcome.
[This zulip discussion](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Composition.20of.20immersions.20is.20an.20immersion.3A.20infinite-dimensio/with/507300190) contains a proof of the non-trivial sorry.
[](https://gitpod.io/from-referrer/)
|
t-analysis
WIP
help-wanted
|
249/0 |
Mathlib.lean,Mathlib/Analysis/NormedSpace/HahnBanach/Splits.lean |
2 |
1 |
['github-actions'] |
nobody |
85-44839 2 months ago |
85-44866 2 months ago |
0-0 0 seconds |
26115 |
grunweg author:grunweg |
WIP/proof of concept,feat: the inverse function theorem for manifolds |
---
[](https://gitpod.io/from-referrer/)
|
t-differential-geometry
WIP
|
348/0 |
Mathlib.lean,Mathlib/Analysis/Calculus/ContDiff/Defs.lean,Mathlib/Geometry/Manifold/InverseFunctionTheorem.lean,Mathlib/Topology/PartialHomeomorph.lean |
4 |
1 |
['github-actions'] |
nobody |
85-43776 2 months ago |
86-60242 2 months ago |
0-0 0 seconds |
25803 |
erdOne author:erdOne |
feat: taylor expansion of `1 / z ^ r` |
---
This might exist somewhere else but I couldn't find them.
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #21693.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/21693* |
t-analysis
awaiting-author
|
95/0 |
Mathlib.lean,Mathlib/Analysis/SpecificLimits/InvPow.lean |
2 |
5 |
['erdOne', 'github-actions', 'j-loreaux', 'vasnesterov'] |
nobody |
84-51854 2 months ago |
84-51854 2 months ago |
8-29520 8 days |
26239 |
BoltonBailey author:BoltonBailey |
feat: add sample pre-commit git hook file |
This PR adds a sample pre-commit git hook file that runs `mk_all` and `lint-style`. The script provides instructions on how to activate these as git hooks. Installing these would be optional, but hopefully people who would install them would find it easier to avoid commits that immediately fail linters.
Discussion of hooks on [Zulip here](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Automatic.20setup.20and.20distribution.20of.20git.20hooks/with/525103090).
Some thoughts:
- Perhaps it would be better, for speed, to attempt to avoid certain commands if the staged changes suggest they would be unnecessary.
- i.e. only run linters on files that have been updated / only run `mk_all` if a file has been added or deleted.
---
[](https://gitpod.io/from-referrer/)
|
WIP |
18/0 |
git_hooks/pre-commit |
1 |
1 |
['github-actions'] |
nobody |
84-48056 2 months ago |
84-48056 2 months ago |
0-1331 22 minutes |
26231 |
chrisflav author:chrisflav |
feat(CategoryTheory/Sites): sheaf condition and coproducts |
We show that under suitable conditions, checking that a presheaf is a sheaf for a covering is equivalent to checking it on the single object covering by the coproduct.
---
I am not sure this is the correct file, but I had no better idea. Happy to move it somewhere else.
[](https://gitpod.io/from-referrer/)
|
t-category-theory
awaiting-author
|
58/0 |
Mathlib/CategoryTheory/Sites/Sheaf.lean |
1 |
3 |
['chrisflav', 'github-actions', 'joelriou'] |
nobody |
83-3685 2 months ago |
83-4343 2 months ago |
1-60053 1 day |
25603 |
callesonne author:callesonne |
feat(Bicategory/InducedBicategory): add induced bicategories |
This PR adds a way of inducing a full bicategory structure on given type of objects with a map to the objects of some bicategory (i.e. with all 1-morphisms and all 2-morphisms).
I have not tried to implement "locally induced bicategories" which should allow for a sub-class of 1-morphisms as well. This is because copying the naive approach and replacing the map `F` as for induced categories with a functor, one runs into issues when the equalities in `F.map_comp` and `F.map_id` are not defeq equalities. One could probably define locally full sub-bicategories using a pair of `ObjectProperty` + `MorphismProperty` to ensure that the inclusions are actually defeq, but I did not want to get into this.
---
[](https://gitpod.io/from-referrer/)
|
t-category-theory
awaiting-author
|
68/0 |
Mathlib.lean,Mathlib/CategoryTheory/Bicategory/InducedBicategory.lean |
2 |
5 |
['callesonne', 'github-actions', 'robin-carlier'] |
robin-carlier assignee:robin-carlier |
82-73476 2 months ago |
83-7127 2 months ago |
13-48345 13 days |
24395 |
rudynicolop author:rudynicolop |
feat(Data/List): list splitting definitions and lemmas |
Adds definitions and lemmas for obtaining all prefixes and suffixes of lists.
---
[](https://gitpod.io/from-referrer/)
|
t-data
new-contributor
awaiting-author
|
143/2 |
Mathlib/Data/List/Perm/Lattice.lean,Mathlib/Data/List/TakeDrop.lean |
2 |
4 |
['BoltonBailey', 'github-actions'] |
ericrbg assignee:ericrbg |
82-45984 2 months ago |
82-45984 2 months ago |
57-9536 57 days |
21450 |
eric-wieser author:eric-wieser |
feat: improve trace nodes for `positivity` |
---
[](https://gitpod.io/from-referrer/)
|
t-meta |
25/7 |
Mathlib/Tactic/Positivity/Core.lean |
1 |
1 |
['github-actions'] |
nobody |
82-44835 2 months ago |
220-15149 7 months ago |
0-0 0 seconds |
26292 |
RemyDegenne author:RemyDegenne |
feat(MeasureTheory): tightness of the range of a sequence |
* `isTightMeasureSet_range_iff_tendsto_limsup_measure_norm_gt`: in a proper normed group,
the range of a sequence of measures `μ : ℕ → Measure E` is tight if and only if the function
`r : ℝ ↦ limsup (fun n ↦ μ n {x | r < ‖x‖}) atTop` tends to `0` at infinity.
* `isTightMeasureSet_range_iff_tendsto_limsup_inner`: in a finite-dimensional inner product space,
the range of a sequence of measures `μ : ℕ → Measure E` is tight if and only if the function
`r : ℝ ↦ limsup (fun n ↦ μ n {x | r < ‖⟪y, x⟫_𝕜‖}) atTop` tends to `0` at infinity for all `y`.
---
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #24838.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/24838* |
t-measure-probability
awaiting-author
|
197/2 |
Mathlib/MeasureTheory/Measure/TightNormed.lean |
1 |
1 |
['github-actions'] |
nobody |
82-7682 2 months ago |
82-7747 2 months ago |
0-1 1 second |
26293 |
RemyDegenne author:RemyDegenne |
feat: tightness from convergence of characteristic functions |
If the characteristic functions of a sequence of measures `μ : ℕ → Measure E` on a finite dimensional inner product space converge pointwise to a function which is continuous at 0, then `{μ n | n}` is tight.
---
- [x] depends on: #24838
- [x] depends on: #24846
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #24949.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/24949* |
t-measure-probability
WIP
|
352/2 |
Mathlib.lean,Mathlib/MeasureTheory/Measure/TightCharFun.lean,Mathlib/MeasureTheory/Measure/TightNormed.lean |
3 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
82-6693 2 months ago |
82-6694 2 months ago |
0-2 2 seconds |
20924 |
tomaz1502 author:tomaz1502 |
feat(Computability/QueryComplexity): Oracle-based computation |
This PR adds the types and lemmas for oracle-based computation. In this model, computations are run on a monad which also counts the number of oracle queries executed. With it, it becomes possible to reason about the upper bound of the query complexity of algorithms. In the future, we could extend this work to include the necessary bits from information theory and probability to also reason about lower bounds on query complexity, like the work in https://github.com/girving/debate.
Zulip discussion: https://leanprover.zulipchat.com/#narrow/channel/144837-PR-reviews/topic/.2318629.20runtime.20complexity.20of.20sorting.20a.20list
Co-authored-by: Geoffrey Irving
---
[](https://gitpod.io/from-referrer/)
|
t-computability |
305/0 |
Mathlib.lean,Mathlib/Computability/QueryComplexity/Basic.lean,Mathlib/Computability/QueryComplexity/Defs.lean |
3 |
59 |
['eric-wieser', 'girving', 'github-actions', 'quangvdao', 'tomaz1502'] |
nobody |
81-72888 2 months ago |
233-66076 7 months ago |
233-66061 233 days |
26327 |
eric-wieser author:eric-wieser |
chore: split the tests for positivity |
---
[](https://gitpod.io/from-referrer/)
|
|
528/2 |
MathlibTest/Positivity/basic.lean,MathlibTest/positivity.lean |
2 |
1 |
['github-actions'] |
nobody |
81-42852 2 months ago |
81-42941 2 months ago |
0-0 0 seconds |
22089 |
sgouezel author:sgouezel |
feat: composing a continuous multilinear map with continuous linear maps is analytic in both variables |
Also prove that the composition of continuously polynomial functions is continuously polynomial.
---
- [x] depends on: #22102
- [x] depends on: #22789
[](https://gitpod.io/from-referrer/)
|
t-analysis
awaiting-author
|
277/80 |
Mathlib/Analysis/Analytic/CPolynomial.lean,Mathlib/Analysis/Analytic/Composition.lean,Mathlib/Analysis/NormedSpace/Multilinear/Basic.lean,Mathlib/Data/Multiset/DershowitzManna.lean,Mathlib/Order/KrullDimension.lean |
5 |
11 |
['github-actions', 'grunweg', 'loefflerd', 'mathlib4-dependent-issues-bot', 'sgouezel', 'urkud'] |
loefflerd assignee:loefflerd |
81-14055 2 months ago |
81-14055 2 months ago |
122-9676 122 days |
26087 |
grunweg author:grunweg |
feat: a `SliceModel` typeclass for models with corners for embedded submanifolds |
We define a new typeclass to denote a model with corners which "embeds" into another one:
there are an embedding of the underlying topological spaces and a continuous linear inclusion between the normed spaces,
which are compatible with the maps given by the models with corners.
This condition is used for defining smooth (immersed and embedded) submanifolds: for `M` to be a submanifold of `N`,
to boot their models with corners should be slice models. This will be defined in a future PR.
To prove this definition is workable, we construct many basic instances of slice models
- each model with corners is one over itself
- slice models are transitive
- each model with corners I embeds into two products `I.prod J` and `J.prod I`
- Euclidean n-half-space embeds into Euclidean n-space
- a Euclidean n-quadrant embeds into Euclidean half-space (hence into Euclidean n-space)
- if n\leq m, Euclidean n-space embeds into Euclidean m-space
[zulip discussion](https://leanprover.zulipchat.com/#narrow/channel/116395-maths/topic/Infinite-dimensional.20manifolds/near/413117885)
-----------
- [x] depends on: #26083
- [x] depends on: #26082
- [x] depends on: #26086
- [x] depends on: #25705
This PR continues the work from #25505. |
t-differential-geometry |
229/0 |
Mathlib.lean,Mathlib/Geometry/Manifold/SliceModel.lean |
2 |
3 |
['github-actions', 'grunweg', 'mathlib4-dependent-issues-bot'] |
nobody |
80-57353 2 months ago |
80-68033 2 months ago |
80-69493 80 days |
26389 |
jjdishere author:jjdishere |
feat(RingTheory): Perfectoid Field |
This PR continues the work from #19972.
Original PR: https://github.com/leanprover-community/mathlib4/pull/19972 |
t-algebra
t-analysis
t-topology
WIP
label:t-algebra$ |
150/0 |
Mathlib/RingTheory/Perfectoid.lean |
1 |
2 |
['github-actions', 'jjdishere'] |
nobody |
80-27396 2 months ago |
80-27403 2 months ago |
0-69 1 minute |
26390 |
jjdishere author:jjdishere |
feat(Topology/Algebra): Krasner's lemma |
This PR continues the work from #18444.
Original PR: https://github.com/leanprover-community/mathlib4/pull/18444 |
t-algebra
t-topology
t-number-theory
WIP
label:t-algebra$ |
440/0 |
Mathlib.lean,Mathlib/Topology/Algebra/Krasner.lean |
2 |
n/a |
['github-actions', 'jjdishere'] |
nobody |
80-27189 2 months ago |
unknown |
unknown |
26376 |
maddycrim author:maddycrim |
Simons2025 |
---
[](https://gitpod.io/from-referrer/)
|
large-import
new-contributor
WIP
|
29/0 |
Mathlib/RingTheory/Localization/Pi.lean |
1 |
1 |
['github-actions'] |
faenuccio assignee:faenuccio |
79-71974 2 months ago |
80-50447 2 months ago |
0-13 13 seconds |
26432 |
AntoineChambert-Loir author:AntoineChambert-Loir |
feat(Data.Nat.LogFueled): fueled version of `clog` |
This PR continues the work from #25557.
Original PR: https://github.com/leanprover-community/mathlib4/pull/25557 |
t-data |
201/0 |
Mathlib.lean,Mathlib/Data/Nat/LogFueled.lean |
2 |
2 |
['AntoineChambert-Loir', 'github-actions'] |
nobody |
79-928 2 months ago |
79-930 2 months ago |
79-979 79 days |
25739 |
literandltx author:literandltx |
feat(NumberTheory/LegendreSymbol): Add sqrt‐of‐residue theorems for p=4k+3 and p=8k+5 |
Add a new file `QuadraticResidueRoots.lean` under `Mathlib/NumberTheory/LegendreSymbol/` that proves two explicit “square-root of quadratic residue” theorems for primes of the specific form.
- **`exists_sqrt_of_residue_mod4_eq3`** for primes `p = 4*k + 3`
- **`exists_sqrt_of_residue_mod8_eq5`** for primes `p = 8*k + 5`
It also introduces the helper lemmas `euler_criterion_traditional` and `legendreSym.at_two_mod8_eq_5`. Import lines in `Mathlib.lean` and `Mathlib/NumberTheory/LegendreSymbol/Basic.lean` have been updated accordingly.
|
new-contributor
t-number-theory
awaiting-author
|
217/0 |
Mathlib.lean,Mathlib/NumberTheory/LegendreSymbol/Basic.lean,Mathlib/NumberTheory/LegendreSymbol/QuadraticReciprocity.lean,Mathlib/NumberTheory/LegendreSymbol/QuadraticResidueRoots.lean |
4 |
2 |
['github-actions', 'kckennylau'] |
literandltx assignee:literandltx |
75-5101 2 months ago |
75-34187 2 months ago |
17-63153 17 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
awaiting-author
label:t-algebra$ |
27/10 |
Mathlib/Algebra/Group/Units/Basic.lean,Mathlib/Algebra/Group/Units/Hom.lean |
2 |
5 |
['Multramate', 'Ruben-VandeVelde', 'github-actions'] |
nobody |
74-6853 2 months ago |
74-6853 2 months ago |
14-37502 14 days |
26013 |
tsuki8 author:tsuki8 |
feat(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
---
[](https://gitpod.io/from-referrer/)
|
t-data
new-contributor
awaiting-author
|
15/0 |
Mathlib/Data/Finset/Card.lean,Mathlib/Data/Set/Finite/Basic.lean |
2 |
5 |
['Ruben-VandeVelde', 'github-actions'] |
nobody |
73-79876 2 months ago |
74-5768 2 months ago |
13-85893 13 days |
26348 |
mans0954 author:mans0954 |
WIP: feature(Analysis/LocallyConvex/Prime): The prime map |
This PR continues the work from #24385.
Original PR: https://github.com/leanprover-community/mathlib4/pull/24385 |
t-analysis
WIP
|
125/0 |
Mathlib.lean,Mathlib/Analysis/LocallyConvex/Prime.lean |
2 |
2 |
['github-actions', 'mans0954'] |
nobody |
72-50326 2 months ago |
75-54557 2 months ago |
5-43062 5 days |
26346 |
mans0954 author:mans0954 |
feature(LinearAlgebra/QuadraticForm/TensorProduct): Extend `baseChange_ext` to work over a free module |
This PR continues the work from #21814.
Original PR: https://github.com/leanprover-community/mathlib4/pull/21814 |
t-algebra
WIP
label:t-algebra$ |
105/5 |
Mathlib/LinearAlgebra/Basis/Bilinear.lean,Mathlib/LinearAlgebra/QuadraticForm/TensorProduct.lean |
2 |
2 |
['github-actions', 'mans0954'] |
nobody |
72-50250 2 months ago |
75-54381 2 months ago |
0-0 0 seconds |
26283 |
kckennylau author:kckennylau |
(WIP) Resultant |
---
This is a WIP PR for resultant for me to get cache.
PRs produced:
* [x] #25139
(migrated to #26091)
* [x] #25270
* [x] #25279
* [x] #25293
* [x] #25294
* [x] #25305
* [x] #26285
[](https://gitpod.io/from-referrer/)
|
t-algebra
WIP
label:t-algebra$ |
1190/0 |
Mathlib.lean,Mathlib/Algebra/Polynomial/Resultant/Basic.lean,Mathlib/Algebra/Polynomial/Resultant/MvPolynomial.lean,Mathlib/RingTheory/Polynomial/Discriminant.lean |
4 |
1 |
['github-actions'] |
nobody |
72-34781 2 months ago |
82-22198 2 months ago |
0-19 19 seconds |
26743 |
grunweg author:grunweg |
WIP: product rule for Lie bracket on manifolds |
On the path towards geodesics and the Levi-Civita connection.
---
[](https://gitpod.io/from-referrer/)
|
t-differential-geometry
WIP
|
119/22 |
Mathlib/Geometry/Manifold/VectorField/LieBracket.lean,Mathlib/Geometry/Manifold/VectorField/Pullback.lean |
2 |
1 |
['github-actions'] |
nobody |
70-52937 2 months ago |
70-74411 2 months ago |
0-1 1 second |
16303 |
grunweg author:grunweg |
feat(CI): check for badly formatted titles or missing/contradictory labels |
---
The zulip workflow is entirely cargo-culted from #16296; please review carefully.
[](https://gitpod.io/from-referrer/)
|
CI
awaiting-author
|
325/0 |
.github/build.in.yml,Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter/ValidatePRTitle.lean,MathlibTest/ValidatePRTitle.lean,lakefile.lean,scripts/README.md,scripts/check-title-labels.lean |
8 |
44 |
['Command-Master', 'adomani', 'bryangingechen', 'edegeltje', 'github-actions', 'grunweg', 'joneugster', 'leanprover-community-bot-assistant'] |
bryangingechen assignee:bryangingechen |
70-24388 2 months ago |
70-24388 2 months ago |
78-54824 78 days |
20784 |
eric-wieser author:eric-wieser |
fix: prevent `exact?` recursing forever on `n = 55` |
Test case thanks to @llllvvuu:
```lean
import Mathlib.SetTheory.Ordinal.Basic
theorem natCast_inj {m n : ℕ} : (m : Ordinal) = n ↔ m = n := sorry
example (n : Nat) : n = 55 := by
exact?
```
This is surely a workaround for some unreported lean bug. The bug still exists for `n = 71` or higher, so we can still track down the bug after merging this patch.
---
[](https://gitpod.io/from-referrer/)
|
t-set-theory |
22/3 |
Mathlib/SetTheory/Ordinal/Basic.lean,MathlibTest/LibrarySearchRecDepth.lean |
2 |
15 |
['Command-Master', 'eric-wieser', 'github-actions', 'kbuzzard', 'kim-em', 'leanprover-bot', 'leanprover-community-bot-assistant', 'mattrobball'] |
nobody |
69-78309 2 months ago |
69-78344 2 months ago |
102-65615 102 days |
26561 |
b-mehta author:b-mehta |
feat(LiminfLimsup): liminf of an antitone function is its supremum |
---
[](https://gitpod.io/from-referrer/)
- [x] depends on: #26560 |
t-topology |
24/0 |
Mathlib/Topology/Order/LiminfLimsup.lean |
1 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
68-54337 2 months ago |
68-54548 2 months ago |
0-6 6 seconds |
26449 |
faenuccio author:faenuccio |
feat(NumberTheory/LocalFields/Basic): provide the definition of (valued) Local Field |
In this PR we give the first definition of a local field, scoped in the namespace `Valued`, as a field endowed with a `Valued` structure such that the valuation is discrete, it is complete with respect to the topology induced by the valuation, and the residue field is finite. In future PR's we'll provide an analogous charcterizations (in purely topological terms) and the theory of extensions of local fields.
A first version was in #23730, now closed.
Co-authored-by: María Inés de Frutos-Fernández @mariainesdff
- [x] depends on: #23727
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-number-theory
WIP
label:t-algebra$ |
78/0 |
Mathlib.lean,Mathlib/NumberTheory/LocalFields/Basic.lean |
2 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
68-4469 2 months ago |
68-4476 2 months ago |
0-91 1 minute |
26878 |
adomani author:adomani |
feat: declaration diff script in Lean |
Although, it is still text-based, the parsing of the output of `git diff` is now done in Lean.
The new script already performed better than the old one in a couple of situations:
* #26877
See [this comment](https://github.com/leanprover-community/mathlib4/pull/26847#issuecomment-3045308885)
* #26849
See [this comment](https://github.com/leanprover-community/mathlib4/pull/26849#issuecomment-3045092965)
---
This is still work in progress: the parsing should be more or less done, but I have not yet hooked this into the action workflow.
[](https://gitpod.io/from-referrer/)
|
|
497/0 |
scripts/DeclarationDiff_text_based.lean |
1 |
4 |
['adomani', 'bryangingechen', 'github-actions'] |
bryangingechen assignee:bryangingechen |
67-6436 2 months ago |
67-56387 2 months ago |
0-0 0 seconds |
26990 |
joelriou author:joelriou |
feat(CategoryTheory/Abelian): Noetherian objects form a Serre class |
This PR continues the work from #22367.
Original PR: https://github.com/leanprover-community/mathlib4/pull/22367 |
t-category-theory
WIP
|
311/14 |
Mathlib.lean,Mathlib/CategoryTheory/Abelian/SerreClass/NoetherianObject.lean,Mathlib/CategoryTheory/Abelian/Subobject.lean,Mathlib/CategoryTheory/Subobject/Basic.lean,Mathlib/CategoryTheory/Subobject/MonoOver.lean |
5 |
1 |
['github-actions'] |
nobody |
63-85081 2 months ago |
63-85100 2 months ago |
0-45 45 seconds |
26994 |
Paul-Lez author:Paul-Lez |
feat(Topology/MetricSpace/Pseudo/Defs): add easy lemma about opens in topological spaces |
Split from #26992
---
[](https://gitpod.io/from-referrer/)
|
t-topology
easy
awaiting-author
|
9/0 |
Mathlib/Topology/MetricSpace/Pseudo/Defs.lean |
1 |
4 |
['Paul-Lez', 'github-actions', 'grunweg'] |
nobody |
63-71493 2 months ago |
63-72915 2 months ago |
0-11233 3 hours |
27069 |
FrankieNC author:FrankieNC |
feat(Analysis/MetricSpace/HausdorffDimension): prove dimH of intervals and segments is 1 |
Add theorems `dimH_Icc01` and `dimH_segment` showing that the Hausdorff dimension of the unit interval [0,1] and of any non-degenerate real segment is 1.
The key idea is that the segment is the image of [0,1] under a bi-Lipschitz map. We explicitly construct this map and prove it is both Lipschitz and antilipschitz, allowing us to transfer the dimension result from the unit interval.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-topology
awaiting-author
|
63/0 |
Mathlib/Topology/MetricSpace/HausdorffDimension.lean |
1 |
10 |
['AntoineChambert-Loir', 'FrankieNC', 'github-actions', 'grunweg'] |
nobody |
61-51926 1 month ago |
61-64410 1 month ago |
0-13398 3 hours |
27135 |
JovanGerb author:JovanGerb |
feat: `gconvert` tactic |
The `gconvert` tactic calls `gcongr` internally, and it can be used as replacement/generalization of `peel`.
One drawback is that `peel` can unfold definitions until they are a binder, while `gconvert` cannot, but I think this is acceptable.
TODO: replace all uses of `peel` with either `gconvert` or `congr!`
---
[](https://gitpod.io/from-referrer/)
|
t-meta |
320/17 |
Mathlib/Tactic/GCongr/Core.lean,MathlibTest/GConvert.lean |
2 |
1 |
['github-actions'] |
nobody |
60-70608 1 month ago |
60-70608 1 month ago |
0-0 0 seconds |
27206 |
grhkm21 author:grhkm21 |
feat(CategoryTheory/Adjunction): partial adjoints are adjoints |
Partial adjunctions `F.partial{Left,Right}Adjunction` are adjunctions when fully
defined i.e. `F.{left,right}AdjointObjIsDefined = ⊤`.
|
t-category-theory |
48/2 |
Mathlib/CategoryTheory/Adjunction/PartialAdjoint.lean |
1 |
1 |
['github-actions'] |
nobody |
58-81278 1 month ago |
58-81296 1 month ago |
58-81328 58 days |
18230 |
digama0 author:digama0 |
feat(Tactic/ScopedNS): extend `scoped[NS]` to more commands |
refactor `ScopedNS` to remove error prone repetitiveness and extend it to other commands such as `syntax`, `macro`, `elab`, etc.
Co-authored-by: Jon Eugster
---
[](https://gitpod.io/from-referrer/)
|
t-meta
awaiting-author
|
201/26 |
Mathlib/Tactic/ScopedNS.lean,MathlibTest/scopedNS.lean |
2 |
7 |
['adomani', 'digama0', 'eric-wieser', 'github-actions', 'joneugster', 'kbuzzard'] |
nobody |
57-85972 1 month ago |
200-85477 6 months ago |
41-32344 41 days |
26338 |
mans0954 author:mans0954 |
feat(Order/ScottContinuity): Scott continuity on product spaces |
Some further results on Scott Continuity:
- `scottContinuous_iff_map_sSup`: `f` is Scott continuous if and only if it commutes with `sSup` on directed sets
- `ScottContinuous_prod_of_ScottContinuous`: `f` is Scott continuous on a product space if it is Scott continuous in each variable
- `ScottContinuousOn.inf₂`: For complete linear orders, the meet operation is Scott continuous
---
- [x] depends on: #13201 - I think this is due to the move of the definition of Scott Continuity into its own file rather than a hard dependency.
- [x] depends on: #19150
- [x] depends on: #19222
- [x] depends on:#20254
- [x] depends on: #21493
Original PR: https://github.com/leanprover-community/mathlib4/pull/15412
[](https://gitpod.io/from-referrer/) |
t-order
awaiting-author
|
132/4 |
Mathlib.lean,Mathlib/Order/Bounds/Basic.lean,Mathlib/Order/ScottContinuity.lean,Mathlib/Order/ScottContinuity/Complete.lean,Mathlib/Order/ScottContinuity/Prod.lean |
5 |
n/a |
['YaelDillies', 'github-actions', 'mans0954', 'mathlib4-dependent-issues-bot'] |
nobody |
57-15523 1 month ago |
unknown |
unknown |
26962 |
themathqueen author:themathqueen |
feat(Data/Nat/Fib/Basic): some API for `Nat.fib` |
Added some helpful lemmas for `Nat.fib`.
---
[](https://gitpod.io/from-referrer/)
|
t-data
new-contributor
awaiting-author
|
24/0 |
Mathlib/Data/Nat/Fib/Basic.lean |
1 |
7 |
['Ruben-VandeVelde', 'github-actions', 'themathqueen', 'vihdzp'] |
nobody |
56-54468 1 month ago |
56-54469 1 month ago |
8-31586 8 days |
27323 |
kckennylau author:kckennylau |
chore: make the arguments of fiberInclusion explicit |
---
[](https://gitpod.io/from-referrer/)
|
t-category-theory |
18/17 |
Mathlib/CategoryTheory/FiberedCategory/Fiber.lean,Mathlib/CategoryTheory/FiberedCategory/HasFibers.lean |
2 |
1 |
['github-actions'] |
nobody |
54-4022 1 month ago |
54-4065 1 month ago |
54-4071 54 days |
27187 |
Komyyy author:Komyyy |
feat: `NONote` represents ordinals < ε₀ |
---
[](https://gitpod.io/from-referrer/)
|
t-set-theory
WIP
|
186/12 |
Mathlib/SetTheory/Ordinal/Notation.lean |
1 |
2 |
['github-actions', 'vihdzp'] |
nobody |
53-36632 1 month ago |
59-27080 1 month ago |
0-2 2 seconds |
27330 |
BoltonBailey author:BoltonBailey |
feat(Tactic/Linter): add TacticMs for natural subtraction and division |
This is a (pair of) short tactic scripts I wrote for Project Numina while vetting formal formal statements (thanks to [this guide](https://github.com/mirefek/lean-tactic-programming-guide) for the primer). The scripts check for the presence of natural subtraction and natural division, which can often lead to mistakes.
Of course, Mathlib allows natural subtraction freely, so it's not obvious this could be made useful to Mathlib itself. Still, maybe it's of use to some other project, so I'll leave it here.
---
[](https://gitpod.io/from-referrer/)
|
t-linter |
66/0 |
Mathlib/Tactic/Linter/TruncatedNat.lean |
1 |
2 |
['BoltonBailey', 'eric-wieser', 'github-actions'] |
nobody |
53-30097 1 month ago |
53-50422 1 month ago |
0-0 0 seconds |
26803 |
bjoernkjoshanssen author:bjoernkjoshanssen |
feat: second partial derivatives test |
We prove that if `f` is a real-valued function on `n`-dimensional Euclidean space with vanishing gradient at `x₀`, having a power series on a ball of positive radius around `x₀`, whose second Frechét derivative is positive definite at `x₀`, then
`f` has local minimum at `x₀`.
This project was started at the Lean for Mathematicians workshop hosted by the Simons Foundation in June 2025 in a group consisting of Bjørn Kjos-Hanssen, Erin Griffin, Asaf Kapota, and Janani Lakshmanan, see repo at https://github.com/bjoernkjoshanssen/secondpartial
---
[](https://gitpod.io/from-referrer/)
|
t-analysis
awaiting-author
|
325/0 |
Mathlib.lean,Mathlib/Analysis/Calculus/PartialDerivativeTest.lean |
2 |
11 |
['bjoernkjoshanssen', 'github-actions', 'j-loreaux', 'themathqueen'] |
nobody |
53-19285 1 month ago |
64-26044 2 months ago |
5-11006 5 days |
12006 |
adomani author:adomani |
feat: the `suffa` tactic |
The `suffa` tactic.
`suffa tac` runs the tactic sequence `tac` and returns a `Try this:` suggestion
of the form `suffices [target_after_tac] by tac; assumption`.
For example
```lean
example {m n : Nat} (h : m = n) : 0 + m = n := by
suffa rewrite [Nat.zero_add]
assumption
```
suggests the replacement
```lean
example {m n : Nat} (h : m = n) : 0 + m = n := by
suffices m = n by
rewrite [Nat.zero_add]
assumption
assumption
```
See [this thread](https://leanprover.zulipchat.com/#narrow/stream/113488-general/topic/Try.20this.3A.20suffices.20simpa) as well as [this message](https://leanprover.zulipchat.com/#narrow/stream/144837-PR-reviews/topic/.2311822.20flexible.20tactics.20linter/near/431895664).
---
[](https://gitpod.io/from-referrer/)
|
t-meta
awaiting-author
|
161/0 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Suffa.lean,test/Suffa.lean |
4 |
3 |
['MoritzBeroRoos', 'YaelDillies'] |
nobody |
51-61059 1 month ago |
463-83299 1 year ago |
58-85902 58 days |
27435 |
callesonne author:callesonne |
feat(Normed/Algebra/Logarithm): add FormalMultilinearSeries of logarithm around `1` |
This PR adds the `FormalMultilinearSeries` corresponding to `log` around `1` (or rather, corresponding to `log(1 + x)`. For now, this PR just adds the definition, and copies over as many (easy) results as possible from the corresponding exponential file.
In a follow up PR, we will add a criterion for when the logarithm converges on the unit disk (based on the growth of the inverse norms of naturals in the given algebra), and show that this holds for any Q_p algebra.
This work has been done as part of the workshop "Formalizing Class Field Theory" in Oxford.
Since much of this is copy-pasting the Exponential file, I have kept Anatole Dedecker and Eric Wieser as coauthors.
---
[](https://gitpod.io/from-referrer/)
|
t-analysis
WIP
|
311/0 |
Mathlib/Analysis/Normed/Algebra/Logarithm.lean |
1 |
1 |
['github-actions'] |
nobody |
50-67205 1 month ago |
50-67543 1 month ago |
0-29 29 seconds |
26393 |
winstonyin author:winstonyin |
feat: solutions to $C^n$ vector fields are $C^n$ in time |
I prove that solutions to $C^n$ vector fields are also $C^n$ in time, where $n ≤ \infty$.
This PR continues the work from #21286.
---
- [x] depends on: #26392 [technically only depends on #26382 but I'm writing these as incremental PRs]
[](https://gitpod.io/from-referrer/)
|
t-dynamics
t-analysis
awaiting-author
|
93/2 |
Mathlib/Analysis/Calculus/Deriv/Basic.lean,Mathlib/Analysis/ODE/PicardLindelof.lean |
2 |
19 |
['github-actions', 'grunweg', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'winstonyin'] |
grunweg assignee:grunweg |
50-7583 1 month ago |
50-7583 1 month ago |
2-8489 2 days |
27434 |
plp127 author:plp127 |
test: `AlgEquiv.inv_apply` |
For testing a new `@[simp]` lemma.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
20/1 |
Mathlib/Algebra/Algebra/Equiv.lean,Mathlib/Algebra/Group/End.lean,Mathlib/Algebra/Module/Equiv/Basic.lean,Mathlib/FieldTheory/KrullTopology.lean |
4 |
6 |
['eric-wieser', 'github-actions', 'plp127'] |
nobody |
49-85389 1 month ago |
50-67669 1 month ago |
0-0 0 seconds |
21915 |
YaelDillies author:YaelDillies |
feat: simproc for `Int.divisorsAntidiag` |
Co-authored-by: Paul Lezeau
---
- [x] depends on: #21912
- [x] depends on: #21991
[](https://gitpod.io/from-referrer/)
|
t-meta
WIP
|
73/0 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Simproc/DivisorsAntidiag.lean |
3 |
8 |
['YaelDillies', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
49-74436 1 month ago |
49-74455 1 month ago |
0-260 4 minutes |
26196 |
adomani author:adomani |
fix: silence commandStart on attribute |
This is only a temporary fix, the linter should be able to ignore more granularly individual attributes.
Note: this PR is prompted by "future" changes to mathlib and may not be needed after all!
See [Zulip](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/commandStart.20linter.20broken.20with.20.60grind.60/with/524980336) and also [#mathlib4 > `grind` is available. What should Mathlib users expect? @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/.60grind.60.20is.20available.2E.20What.20should.20Mathlib.20users.20expect.3F/near/526547091) and [lean4#9128](https://github.com/leanprover/lean4/pull/9128) that should be the final attempt to resolve pretty-printing of `grind`, instead of silencing the linter.
---
[](https://gitpod.io/from-referrer/)
|
t-linter |
9/0 |
Mathlib/Tactic/Linter/CommandStart.lean,MathlibTest/CommandStart.lean |
2 |
3 |
['adomani', 'github-actions', 'grunweg'] |
kim-em assignee:kim-em |
49-43554 1 month ago |
85-17198 2 months ago |
0-0 0 seconds |
27507 |
grunweg author:grunweg |
wip(commandStart): check the indentation of declaration keywords also |
Check that e.g. a `lemma` keyword always starts on column 1 (unless preceded by an attribute).
---
TODO:
- make this work for other declarations also
- the position reported for the lemma column is not helpful (it might be the absolute column in the file, but that's missing line information)
[](https://gitpod.io/from-referrer/)
|
t-linter
WIP
|
84/1 |
Mathlib/Tactic/Linter/CommandStart.lean,MathlibTest/CommandStart.lean |
2 |
2 |
['github-actions', 'grunweg'] |
nobody |
48-84438 1 month ago |
48-84509 1 month ago |
0-2 2 seconds |
26594 |
metakunt author:metakunt |
feat(Algebra/Polynomial/ZMod): Add Polynomial.equiv_of_nat_of_polynomial_zmod |
This adds an explicit bijection between the naturals and $$\mathbb{Z}/n\mathbb{Z}[X]$$ in a canonical way.
---
I feel that some API is missing to make the theorem shorter, I have no idea what lemmas to extract though.
Also I don't know when to use spaces and when not, so I did it best effort.
|
new-contributor
t-algebra
awaiting-author
label:t-algebra$ |
465/0 |
Mathlib.lean,Mathlib/Algebra/Polynomial/ZMod.lean |
2 |
2 |
['Ruben-VandeVelde', 'github-actions'] |
nobody |
48-54022 1 month ago |
48-54022 1 month ago |
25-6199 25 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
t-linter
maintainer-merge
awaiting-author
|
375/7 |
Mathlib.lean,Mathlib/Analysis/Meromorphic/FactorizedRational.lean,Mathlib/CategoryTheory/Comma/StructuredArrow/CommaMap.lean,Mathlib/Init.lean,Mathlib/RepresentationTheory/Homological/GroupHomology/LowDegree.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter/EmptyLine.lean,MathlibTest/EmptyLine.lean |
8 |
12 |
['adomani', 'bryangingechen', 'eric-wieser', 'github-actions'] |
bryangingechen assignee:bryangingechen |
46-72751 1 month ago |
46-72751 1 month ago |
42-26074 42 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
awaiting-author
|
151/0 |
.github/workflows/PR_summary_lean.yml,scripts/README.md,scripts/declarations_diff.lean,scripts/declarations_diff_lean_shell_glue.sh |
4 |
7 |
['bryangingechen', 'github-actions', 'grunweg', 'j-loreaux'] |
robertylewis assignee:robertylewis |
46-40079 1 month ago |
46-40079 1 month ago |
146-23504 146 days |
27422 |
vihdzp author:vihdzp |
feat: relate images to pointwise negation/inverses |
These lemmas kept coming up in the CGT repo.
---
[](https://gitpod.io/from-referrer/)
|
t-data
t-algebra
awaiting-author
label:t-algebra$ |
13/0 |
Mathlib/Algebra/Group/Pointwise/Set/Basic.lean |
1 |
7 |
['YaelDillies', 'github-actions', 'vihdzp'] |
nobody |
46-27335 1 month ago |
46-27335 1 month ago |
4-29607 4 days |
26307 |
j-loreaux author:j-loreaux |
refactor: make `IsIdempotentElem` a one-field structure |
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebra
label:t-algebra$ |
29/22 |
Mathlib/Algebra/Group/Idempotent.lean,Mathlib/Algebra/Group/Submonoid/Membership.lean,Mathlib/Algebra/GroupWithZero/Idempotent.lean,Mathlib/Algebra/Ring/BooleanRing.lean,Mathlib/Algebra/Ring/Idempotent.lean |
5 |
1 |
['github-actions'] |
nobody |
45-58976 1 month ago |
81-69516 2 months ago |
0-0 0 seconds |
27677 |
jkpjkpjkp author:jkpjkpjkp |
extend tactic `observe` as syntax sugar for `grind` |
---
The `observe` tactic now attempts to use the `grind` tactic as a fallback
when library search (exact?) fails.
cc. https://leanprover.zulipchat.com/#narrow/channel/113488-general/topic/.22Missing.20Tactics.22.20list/near/531764184
this drafty version does not update doc or `observe?`, as details and decisions may need further discussion. |
new-contributor
t-meta
|
31/8 |
Mathlib/Tactic/Observe.lean |
1 |
2 |
['euprunin', 'github-actions'] |
nobody |
43-52654 1 month ago |
44-85902 1 month ago |
0-0 0 seconds |
27297 |
hugh-fox author:hugh-fox |
feat: add an equality between sums and products of cartesian products |
Adds `prod_mul_eq_prod_product` and a version for Finsets `prod_range_mul_eq_prod_product` with to show an equality between `Fin (i * j)` and `Fin a × Fin b`.
It is likely `prod_range_mul_eq_prod_product` belongs in a different file, in which case only the first commit should be considered.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-algebra
awaiting-author
label:t-algebra$ |
12/0 |
Mathlib/Algebra/BigOperators/Fin.lean |
1 |
6 |
['Ruben-VandeVelde', 'github-actions', 'hugh-fox', 'j-loreaux', 'kckennylau'] |
nobody |
44-54546 1 month ago |
48-46534 1 month ago |
7-6727 7 days |
25864 |
plp127 author:plp127 |
feat(Nat/Digits): use fuel in `Nat.digits` |
Add a `fuel` parameter to `Nat.digitsAux` to make it structurally recursive.
---
[](https://gitpod.io/from-referrer/)
|
t-data |
47/14 |
Mathlib/Data/Nat/Digits/Defs.lean |
1 |
2 |
['github-actions', 'leanprover-community-bot-assistant'] |
ericrbg assignee:ericrbg |
44-54084 1 month ago |
55-44760 1 month ago |
76-4915 76 days |
27704 |
vihdzp author:vihdzp |
feat: link `Minimal` and `IsLeast` together |
---
[](https://gitpod.io/from-referrer/)
|
t-order
awaiting-author
|
24/0 |
Mathlib/Order/Bounds/Basic.lean |
1 |
3 |
['b-mehta', 'github-actions'] |
nobody |
43-78851 1 month ago |
43-78851 1 month ago |
0-52136 14 hours |
14237 |
js2357 author:js2357 |
feat: Define the localization of a fractional ideal at a prime ideal |
Define the localization of a fractional ideal at a prime ideal, and prove some basic properties.
---
This PR is part 3 out of 4 of a proof of `isDedekindDomain_iff_isDedekindDomainDvr`.
Part 4 is available here: #14242
- [x] depends on: #14099 Part 1
- [x] depends on: #14216 Part 2
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-algebra
awaiting-author
label:t-algebra$ |
230/0 |
Mathlib.lean,Mathlib/RingTheory/FractionalIdeal/LocalizedAtPrime.lean,Mathlib/RingTheory/Localization/Basic.lean |
3 |
21 |
['Vierkantor', 'YaelDillies', 'github-actions', 'js2357', 'kbuzzard', 'leanprover-community-bot-assistant', 'leanprover-community-mathlib4-bot'] |
Vierkantor assignee:Vierkantor |
43-64348 1 month ago |
43-64380 1 month ago |
26-39463 26 days |
27756 |
grunweg author:grunweg |
feat: `Weak(Pseudo)EMetricSpace`, generalises `(Pseudo)EMetricSpace` |
---
[](https://gitpod.io/from-referrer/)
|
carleson
t-topology
WIP
|
142/36 |
Mathlib/Topology/EMetricSpace/Defs.lean,Mathlib/Topology/Instances/ENNReal/Lemmas.lean |
2 |
1 |
['github-actions'] |
nobody |
43-47261 1 month ago |
43-68830 1 month ago |
0-2 2 seconds |
27066 |
vasnesterov author:vasnesterov |
feat(Tactic/Order): frontend for `order` |
* Support `order [h1, h2]` and `order only [h1, h2]` syntax.
* Split conjunctions while extracting facts from the context. E.g. hypotheses in the form `A ∧ B` are converted into two facts `A` and `B`.
* Similarly, extract facts from existential quantifiers in the hypotheses.
---
- [x] depends on: #26354
[](https://gitpod.io/from-referrer/)
This PR continues the work from #22073.
Original PR: https://github.com/leanprover-community/mathlib4/pull/22073 |
t-meta |
91/37 |
Mathlib.lean,Mathlib/Tactic/Linarith/Frontend.lean,Mathlib/Tactic/Order.lean,Mathlib/Tactic/Order/CollectFacts.lean,Mathlib/Util/ElabWithoutMVars.lean,MathlibTest/order.lean |
6 |
22 |
['JovanGerb', 'github-actions', 'mathlib4-dependent-issues-bot', 'vasnesterov'] |
alexjbest assignee:alexjbest |
43-44555 1 month ago |
62-4482 2 months ago |
62-4507 62 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
awaiting-author
|
259/37 |
Mathlib/NumberTheory/EllipticDivisibilitySequence.lean |
1 |
8 |
['MichaelStollBayreuth', 'Multramate', 'github-actions', 'tb65536'] |
tb65536 assignee:tb65536 |
43-43731 1 month ago |
43-43731 1 month ago |
45-1019 45 days |
27813 |
javra author:javra |
feat: IMO 2025 Q1 |
---
[](https://gitpod.io/from-referrer/)
|
IMO
WIP
|
882/0 |
Archive/Imo/Imo2025Q1.lean |
1 |
1 |
['github-actions'] |
nobody |
42-82632 1 month ago |
42-83830 1 month ago |
0-14 14 seconds |
22366 |
kim-em author:kim-em |
feat: `check_equalities` tactic for diagnosing defeq problems |
The `check_equalities` tactic,
which checks the typing of equalities in the goal,
reporting discrepancies between the implicit type argument of the equality,
and the inferred types of the left and right hand sides,
at "instances and reducible" transparency.
Reports from this tactic do not necessarily indicate a problem,
although typically `simp` should reduce rather than increase the reported discrepancies.
`check_equalities` may be useful in diagnosing uses of `erw`. |
t-meta
delegated
|
118/3 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Basic.lean,Mathlib/Tactic/CategoryTheory/CheckCompositions.lean,Mathlib/Tactic/CheckEqualities.lean,Mathlib/Tactic/Common.lean,MathlibTest/check_equalities.lean |
7 |
16 |
['adomani', 'b-mehta', 'eric-wieser', 'github-actions', 'grunweg', 'kim-em', 'mathlib-bors'] |
nobody |
42-77768 1 month ago |
182-70337 5 months ago |
15-14325 15 days |
27683 |
dupuisf author:dupuisf |
feat: grind tags for set operations |
This PR adds `grind` tags for various set operations (union, intersection, complement, etc).
---
[](https://gitpod.io/from-referrer/)
|
t-data |
29/9 |
Mathlib/Data/Set/Basic.lean,Mathlib/Data/Set/Operations.lean |
2 |
4 |
['dupuisf', 'euprunin', 'github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
42-71768 1 month ago |
42-71798 1 month ago |
44-44885 44 days |
27753 |
YunkaiZhang233 author:YunkaiZhang233 |
feat(CategoryTheory): implemented proofs for factorisation categories being equivalent to iterated comma categories in two ways |
---
Completed one of the tasks in TODOs, shown and implemented the details for (X/C)/f ≌ Factorisation f ≌ f/(C/Y).
This is migrated from my previous PR #22390
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-category-theory
awaiting-author
|
70/1 |
Mathlib/CategoryTheory/Category/Factorisation.lean |
1 |
12 |
['YunkaiZhang233', 'b-mehta', 'github-actions', 'robin-carlier'] |
nobody |
42-71749 1 month ago |
43-67630 1 month ago |
0-3448 57 minutes |
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
delegated
label:t-algebra$ |
33/6 |
Mathlib/RingTheory/TensorProduct/Basic.lean |
1 |
7 |
['adomani', 'github-actions', 'kbuzzard', 'leanprover-bot', 'mathlib-bors'] |
adomani assignee:adomani |
42-69961 1 month ago |
42-77090 1 month ago |
56-85445 56 days |
27829 |
dupuisf author:dupuisf |
feat: modify `cfc_tac` to use `grind` |
---
[](https://gitpod.io/from-referrer/)
|
WIP |
60/50 |
Mathlib/Algebra/Order/Star/Basic.lean,Mathlib/Algebra/Star/SelfAdjoint.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Integral.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/NonUnital.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Unital.lean,Mathlib/Analysis/SpecialFunctions/ContinuousFunctionalCalculus/ExpLog.lean,Mathlib/Analysis/SpecialFunctions/ContinuousFunctionalCalculus/PosPart/Basic.lean,Mathlib/Analysis/SpecialFunctions/ContinuousFunctionalCalculus/Rpow/Basic.lean,Mathlib/Tactic/ContinuousFunctionalCalculus.lean |
9 |
1 |
['github-actions'] |
nobody |
42-69861 1 month ago |
42-72359 1 month ago |
0-1 1 second |
25974 |
scholzhannah author:scholzhannah |
feat(Topology/Compactness/CompactlyCoherentSpace): compact coherentification (k-ification) |
This PR defines the notion of turning an arbitrary topological space into a compactly coherent space. Compactly coherent spaces are commonly referred to as "compactly generated spaces" or "k-spaces" in the literature while the operation of turning a space into such as space is called the "k-ification". There are however three different notions that are described with this name. To disambiguate we use the names "compactly coherent space" and "compactcoherentification" here. See [this wikipedia page](https://en.wikipedia.org/wiki/Compactly_generated_space) for an explanation of these notions.
This PR continues the work from #25318.
Original PR: https://github.com/leanprover-community/mathlib4/pull/25318
Co-authored-by: Floris van Doorn |
large-import
t-topology
|
175/5 |
Mathlib/Topology/Compactness/CompactlyCoherentSpace.lean |
1 |
2 |
['github-actions', 'scholzhannah'] |
ADedecker assignee:ADedecker |
42-64610 1 month ago |
88-53176 2 months ago |
88-53221 88 days |
27826 |
Louddy author:Louddy |
feat(Subsemiring): mk_eq_zero |
Add a `mk_eq_zero` lemma for `Subsemiring`.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
WIP
label:t-algebra$ |
4/0 |
Mathlib/Algebra/Ring/Subsemiring/Defs.lean |
1 |
3 |
['Louddy', 'eric-wieser', 'github-actions'] |
nobody |
42-64114 1 month ago |
42-67196 1 month ago |
0-8982 2 hours |
25758 |
YaelDillies author:YaelDillies |
chore: shortcut instance `CompleteLattice α → PartialOrder α` |
This avoids using the path `CompleteLattice α → CompletePartialOrder α → PartialOrder α` that goes through `Order.CompletePartialOrder` and makes it appear used to our automation, such as `shake` or `#min_imports`.
This is a followup to #25358.
---
[](https://gitpod.io/from-referrer/)
|
t-order |
7/0 |
Mathlib/Order/CompleteLattice/Defs.lean |
1 |
6 |
['Ruben-VandeVelde', 'eric-wieser', 'github-actions', 'leanprover-bot'] |
bryangingechen assignee:bryangingechen |
42-34917 1 month ago |
73-42657 2 months ago |
93-6839 93 days |
27050 |
BoltonBailey author:BoltonBailey |
doc(Control/Monad/Cont): add docstrings |
Split of #25917. Adds docstrings to this file. Note: this documentation was written by asking Cursor (Claude 3.5 sonnet) to write the docstrings.
---
[](https://gitpod.io/from-referrer/)
|
t-data
awaiting-author
|
183/0 |
Mathlib/Control/Monad/Cont.lean |
1 |
8 |
['BoltonBailey', 'eric-wieser', 'github-actions'] |
nobody |
42-26642 1 month ago |
61-44325 1 month ago |
0-85623 23 hours |
25916 |
BoltonBailey author:BoltonBailey |
feat: add `simp` lemma `coeff_eq_zero_of_not_mem_support` |
Adds the forward direction of `not_mem_support_iff` as a simp lemma.
Original PR: https://github.com/leanprover-community/mathlib4/pull/13026 |
t-algebra
awaiting-author
label:t-algebra$ |
4/0 |
Mathlib/Algebra/MvPolynomial/Basic.lean |
1 |
2 |
['BoltonBailey', 'github-actions'] |
nobody |
41-67766 1 month ago |
89-68652 2 months ago |
0-8 8 seconds |
27021 |
grunweg author:grunweg |
feat: custom elaborators for differential geometry |
Add two sets of custom elaborators for differential geometry, to
- infer the model with corners in `MDifferentiable{WithinAt,At,On}` or `ContMDiff{WithinAt,At,On}` expressions from the local context, and provide shorter notation in that setting
- do the same for mfderiv: `mfderiv% f` is shorthand for `mfderiv I J f`; `mfderiv[s] f x` is short for `mfderivWithin I J f s`
- convert a fibre bundle section from a dependent section to a function into the total space, making working with differentiability of sections of fibre bundles less cumbersome
This was [discussed on zulip](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Differential.20geometry.20elaborators.20experiment/with/528035295), to overall broad consensus.
This code has substantial tests and has been tried in the branch in #26221 (uncovering minor issues, but not substantial ones). The implementation itself is of prototype quality and will be cleaned up in the future. Once it is more robust, more differential geometry files can be converted to use it.
Co-authored-by: Patrick Massot
-----------
I agree that merging not fully polished code is not ideal, but propose doing so for two reasons:
- the work in #26221 used these elaborators extensively (to test them). Reverting those changes, merging the code, only to re-apply them is not a good use of time. Merging this PR now enables merging the work in #26221 soon.
- the feature is clearly useful and not going away: in the files that use it, it works well already. Holding off on further adopting, but merging it now seems like a good compromise.
---
[](https://gitpod.io/from-referrer/)
|
t-differential-geometry
t-meta
|
782/0 |
Mathlib.lean,Mathlib/Geometry/Manifold/Elaborators.lean,Mathlib/Geometry/Manifold/Traces.lean,MathlibTest/DifferentialGeometry/Elaborators.lean,scripts/noshake.json |
5 |
4 |
['github-actions', 'grunweg', 'sgouezel'] |
robertylewis assignee:robertylewis |
41-34882 1 month ago |
63-8171 2 months ago |
63-8241 63 days |
27225 |
eric-wieser author:eric-wieser |
refactor(Tactic/Lift): deprecate the third with argument |
We already have a number of tactics where the clearing happens all the time, and you have to opt out with `id h`.
This also fixes a bug where `lift z to Nat with n hn this_is_unused` would silently ignore `this_is_unused`.
---
- [ ] depends on: #27223
[](https://gitpod.io/from-referrer/)
|
t-meta
awaiting-author
|
21/9 |
Mathlib/Tactic/Lift.lean,MathlibTest/lift.lean |
2 |
8 |
['JovanGerb', 'adomani', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'vihdzp'] |
JovanGerb assignee:JovanGerb |
41-30133 1 month ago |
41-77033 1 month ago |
15-64386 15 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 |
2 |
['b-mehta', 'github-actions'] |
joelriou assignee:joelriou |
40-65125 1 month ago |
93-6691 3 months ago |
93-6671 93 days |
25042 |
alreadydone author:alreadydone |
feat(Topology): restriction/extension of Trivialization and composition with Homeomorph |
---
- [x] depends on: #25041
[](https://gitpod.io/from-referrer/)
|
t-topology |
148/2 |
Mathlib/Topology/FiberBundle/Trivialization.lean,Mathlib/Topology/Maps/Basic.lean |
2 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
ADedecker assignee:ADedecker |
40-34894 1 month ago |
60-358 1 month ago |
115-70022 115 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'] |
erdOne assignee:erdOne |
40-34891 1 month ago |
87-36632 2 months ago |
87-36675 87 days |
27703 |
vihdzp author:vihdzp |
feat: `le_of_forall_ne` |
This form of `le_of_forall_lt` is a bit nicer when working with nimbers; they're minimum excludents, so to prove `a ≤ b` you have to prove `b` can't be equal to any smaller `a`!
---
[](https://gitpod.io/from-referrer/)
|
t-order
easy
awaiting-author
|
7/0 |
Mathlib/Order/Basic.lean |
1 |
6 |
['JovanGerb', 'eric-wieser', 'github-actions'] |
nobody |
40-34279 1 month ago |
40-40164 1 month ago |
4-6136 4 days |
27915 |
xroblot author:xroblot |
chore: example of the error `uncaught exception: dependency loop found involving Mathlib!` |
This branch contains a file `Loop.lean` that imports all of Mathlib including itself.
When trying to download the corresponding cache, we get the error message
`
Cannot fetch Mathlib build artifact cache. Command output: uncaught exception: dependency loop found involving Mathlib!
`
---
[](https://gitpod.io/from-referrer/)
|
|
2/0 |
Mathlib.lean,Mathlib/Loop.lean |
2 |
1 |
['github-actions'] |
nobody |
40-32801 1 month ago |
40-33021 1 month ago |
40-33001 40 days |
26347 |
mans0954 author:mans0954 |
feature(Data/Finset/RangeDistance): abs_sub_lt_of_mem_finset_range |
This PR continues the work from #23161.
Original PR: https://github.com/leanprover-community/mathlib4/pull/23161 |
t-data |
30/0 |
Mathlib.lean,Mathlib/Algebra/Order/Group/Unbundled/Abs.lean,Mathlib/Data/Finset/RangeDistance.lean |
3 |
2 |
['github-actions', 'mans0954'] |
alreadydone assignee:alreadydone |
40-1893 1 month ago |
40-1893 1 month ago |
81-11303 81 days |
26341 |
mans0954 author:mans0954 |
feat(LinearAlgebra/QuadraticForm/Basis): Free Tensor product of Quadratic Maps |
This PR continues the work from #19432.
Original PR: https://github.com/leanprover-community/mathlib4/pull/19432 |
large-import
t-algebra
WIP
label:t-algebra$ |
888/0 |
Mathlib.lean,Mathlib/Data/Sym/Sym2/Prod.lean,Mathlib/LinearAlgebra/QuadraticForm/Basis.lean |
3 |
n/a |
['github-actions', 'mans0954'] |
nobody |
40-1884 1 month ago |
unknown |
unknown |
26340 |
mans0954 author:mans0954 |
feat(Algebra/Module/NestAlgebra): Nest algebras |
This PR continues the work from #18705.
Original PR: https://github.com/leanprover-community/mathlib4/pull/18705 |
t-algebra label:t-algebra$ |
184/0 |
Mathlib.lean,Mathlib/Algebra/Module/NestAlgebra.lean,Mathlib/Order/Nest.lean,Mathlib/Order/Preorder/Chain.lean,docs/references.bib |
5 |
2 |
['github-actions', 'mans0954'] |
nobody |
40-1880 1 month ago |
40-1880 1 month ago |
81-12814 81 days |
26298 |
adomani author:adomani |
test: the commandStart linter only acts on modified files. |
Test for #26299: should flag issues in the new file and also in the modified file `Mathlib/Data/Array/Extract.lean`.
---
[](https://gitpod.io/from-referrer/)
|
t-linter
awaiting-author
WIP
|
63/1 |
Mathlib.lean,Mathlib/Data/Array/Extract.lean,Mathlib/New.lean,Mathlib/Tactic/Linter/CommandStart.lean |
4 |
20 |
['adomani', 'bryangingechen', 'github-actions'] |
nobody |
40-1841 1 month ago |
40-1842 1 month ago |
0-0 0 seconds |
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 |
t-ring-theory
awaiting-author
|
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 |
9 |
['Multramate', 'Ruben-VandeVelde', 'github-actions'] |
nobody |
40-1802 1 month ago |
40-1802 1 month ago |
39-76045 39 days |
25986 |
Multramate author:Multramate |
feat(AlgebraicGeometry/EllipticCurve/NumberField/Height): define heights on Weierstrass curves |
This PR continues the work from #15786.
Original PR: https://github.com/leanprover-community/mathlib4/pull/15786 |
t-algebraic-geometry |
650/0 |
Mathlib/AlgebraicGeometry/EllipticCurve/NumberField/Height.lean |
1 |
2 |
['Multramate', 'github-actions'] |
nobody |
40-1790 1 month ago |
40-1790 1 month ago |
0-0 0 seconds |
26342 |
mans0954 author:mans0954 |
WiP: Expansion of the tensor product of quadratic maps over a linear combination |
This PR continues the work from #19806.
Original PR: https://github.com/leanprover-community/mathlib4/pull/19806 |
t-algebra
WIP
label:t-algebra$ |
483/0 |
Mathlib/Data/Sym/Sym2/Prod.lean,Mathlib/LinearAlgebra/QuadraticForm/Basic.lean,Mathlib/LinearAlgebra/QuadraticForm/Basis.lean,Mathlib/LinearAlgebra/QuadraticForm/TensorProduct.lean |
4 |
n/a |
['github-actions', 'mans0954'] |
nobody |
40-1728 1 month ago |
unknown |
unknown |
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
awaiting-author
|
101/4 |
Mathlib/NumberTheory/Divisors.lean |
1 |
36 |
['MichaelStollBayreuth', 'github-actions', 'upobir'] |
mariainesdff assignee:mariainesdff |
39-73576 1 month ago |
39-73576 1 month ago |
46-1067 46 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'] |
PatrickMassot assignee:PatrickMassot |
39-34897 1 month ago |
85-79485 2 months ago |
85-79540 85 days |
27108 |
pechersky author:pechersky |
chore(RingTheory/AdicValuation): golf using WithZero.log |
with helper lemma of how `log` preserves order
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-number-theory
label:t-algebra$ |
15/16 |
Mathlib/Algebra/Order/GroupWithZero/Canonical.lean,Mathlib/RingTheory/DedekindDomain/AdicValuation.lean |
2 |
2 |
['YaelDillies', 'github-actions'] |
mariainesdff assignee:mariainesdff |
39-34893 1 month ago |
60-70551 1 month ago |
60-80339 60 days |
26483 |
metakunt author:metakunt |
feat (RingTheory/RootsOfUnity/PrimitiveRoots) : Add equiv_primitiveRoots_of_coprimePow |
Adds equivalence of r-th primitive roots by a coprime e. |
t-ring-theory
new-contributor
awaiting-author
|
79/0 |
Mathlib/RingTheory/RootsOfUnity/PrimitiveRoots.lean |
1 |
13 |
['Citronhat', 'Ruben-VandeVelde', 'github-actions', 'metakunt'] |
nobody |
39-4050 1 month ago |
39-4050 1 month ago |
28-81831 28 days |
26386 |
jjdishere author:jjdishere |
feat(RingTheory/Perfection): lemmas for `frobeniusEquiv.symm` |
This PR continues the work from #22330.
Original PR: https://github.com/leanprover-community/mathlib4/pull/22330 |
t-ring-theory |
321/5 |
Mathlib.lean,Mathlib/Algebra/Ring/Aut.lean,Mathlib/FieldTheory/Perfect.lean,Mathlib/RingTheory/Perfection.lean,Mathlib/RingTheory/Perfectoid/Untilt.lean,Mathlib/RingTheory/WittVector/Basic.lean,Mathlib/RingTheory/WittVector/Complete.lean,Mathlib/RingTheory/WittVector/TeichmullerSeries.lean |
8 |
7 |
['eric-wieser', 'github-actions', 'jjdishere'] |
nobody |
39-3990 1 month ago |
39-3990 1 month ago |
80-27244 80 days |
26368 |
Whysoserioushah author:Whysoserioushah |
feat(RingTheory/TwoSidedIdeal/SpanAsSum): span of set as finsum |
Co-authored-by: Jujian Zhang
---
Reopened after everything moved to fork (#23320).
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
awaiting-author
|
81/0 |
Mathlib.lean,Mathlib/RingTheory/TwoSidedIdeal/SpanAsSum.lean |
2 |
5 |
['github-actions', 'kckennylau'] |
YaelDillies assignee:YaelDillies |
39-3966 1 month ago |
39-3966 1 month ago |
37-40835 37 days |
26387 |
jjdishere author:jjdishere |
feat(RingTheory/WittVector): the Teichmuller series |
This PR continues the work from #22320.
Original PR: https://github.com/leanprover-community/mathlib4/pull/22320 |
t-ring-theory
awaiting-author
|
204/2 |
Mathlib.lean,Mathlib/Algebra/Ring/Aut.lean,Mathlib/FieldTheory/Perfect.lean,Mathlib/RingTheory/WittVector/Basic.lean,Mathlib/RingTheory/WittVector/Complete.lean,Mathlib/RingTheory/WittVector/TeichmullerSeries.lean |
6 |
2 |
['github-actions', 'jjdishere'] |
nobody |
39-3923 1 month ago |
39-3923 1 month ago |
0-87 1 minute |
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-ring-theory |
120/0 |
Mathlib.lean,Mathlib/RingTheory/GradedAlgebra/Homogeneous/Subsemiring.lean |
2 |
1 |
['github-actions'] |
kim-em assignee:kim-em |
39-3837 1 month ago |
39-3837 1 month ago |
87-58954 87 days |
25616 |
erdOne author:erdOne |
feat(RingTheory/Invariant): residue field extension is finite |
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
awaiting-author
|
51/0 |
Mathlib/FieldTheory/Galois/Basic.lean,Mathlib/RingTheory/Invariant/Basic.lean |
2 |
5 |
['github-actions', 'tb65536'] |
nobody |
39-3779 1 month ago |
39-3779 1 month ago |
10-17744 10 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/)
|
t-ring-theory
toric
|
309/0 |
Mathlib.lean,Mathlib/RingTheory/Bialgebra/GroupLike.lean,Mathlib/RingTheory/Coalgebra/GroupLike.lean,Mathlib/RingTheory/HopfAlgebra/GroupLike.lean |
4 |
42 |
['Julian-Kuelshammer', 'Parcly-Taxel', 'Whysoserioushah', 'YaelDillies', 'erdOne', 'eric-wieser', 'github-actions', 'leanprover-bot', 'mathlib4-dependent-issues-bot', 'smorel394'] |
eric-wieser assignee:eric-wieser |
39-3731 1 month ago |
39-3731 1 month ago |
125-47186 125 days |
14733 |
jjaassoonn author:jjaassoonn |
feat(RingTheory/Flat/CategoryTheory): a module is flat iff tensoring preserves finite limits |
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
awaiting-author
|
99/1 |
Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Basic.lean,Mathlib/Algebra/Category/ModuleCat/Monoidal/RightExact.lean,Mathlib/RingTheory/Flat/CategoryTheory.lean |
4 |
2 |
['github-actions', 'kim-em'] |
nobody |
39-3564 1 month ago |
39-3564 1 month ago |
6-6256 6 days |
14727 |
jjaassoonn author:jjaassoonn |
feat(RingTheory/Flat/CategoryTheory): a flat module has vanishing higher Tor groups |
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
awaiting-author
|
37/1 |
Mathlib/RingTheory/Flat/CategoryTheory.lean |
1 |
3 |
['github-actions', 'kim-em'] |
nobody |
39-3552 1 month ago |
39-3552 1 month ago |
3-28223 3 days |
27309 |
kckennylau author:kckennylau |
feat(CategoryTheory): a presheaf on `CostructuredArrow F d` can be extended to a presheaf on `C` |
---
Depends on:
* [ ] #27321
Zulip: [#Is there code for X? > over category via a functor](https://leanprover.zulipchat.com/#narrow/channel/217875-Is-there-code-for-X.3F/topic/over.20category.20via.20a.20functor/with/529574191)
[](https://gitpod.io/from-referrer/)
|
t-category-theory
WIP
|
218/0 |
Mathlib.lean,Mathlib/CategoryTheory/Comma/Presheaf/LeftExtension.lean |
2 |
3 |
['erdOne', 'github-actions', 'robin-carlier'] |
erdOne assignee:erdOne |
39-266 1 month ago |
39-287 1 month ago |
15-69033 15 days |
27976 |
smmercuri author:smmercuri |
feat: `ramificationIdx` for `NumberField.InfinitePlace` |
This PR continues the work from #24884.
Original PR: https://github.com/leanprover-community/mathlib4/pull/24884 |
t-number-theory
WIP
|
22/0 |
Mathlib/NumberTheory/NumberField/InfinitePlace/Ramification.lean |
1 |
1 |
['github-actions'] |
nobody |
39-52 1 month ago |
39-64 1 month ago |
0-57 57 seconds |
27417 |
PierreQuinton author:PierreQuinton |
feat: add `SigmaCompleteLattice` |
A $\sigma$-complete lattice is a lattice in which every countable subset `s` has a least upper bound and a greatest lower bound, denoted below by `sSup s` and `sInf s`.
This PR adds the classes `SigmaCompleteLattice` as well as some theorems (mainly adapted from `CompleteLattice` and `ConditionallyCompleteLattice`). This is an adaptation of #26318
---
[](https://gitpod.io/from-referrer/)
|
t-order
awaiting-author
|
394/0 |
Mathlib.lean,Mathlib/Order/SigmaCompleteLattice.lean |
2 |
8 |
['PierreQuinton', 'YaelDillies', 'github-actions', 'vihdzp'] |
YaelDillies assignee:YaelDillies |
38-64943 1 month ago |
38-64943 1 month ago |
12-33338 12 days |
27292 |
gasparattila author:gasparattila |
feat: asymptotic cone of a set |
This PR defines the asymptotic cone of a set in a normed affine space and proves its main properties. This is partial progress towards showing that an unbounded finite-dimensional convex set contains a ray.
---
- [x] depends on: #27221
[](https://gitpod.io/from-referrer/)
|
maintainer-merge
new-contributor
t-analysis
|
453/0 |
Mathlib.lean,Mathlib/Analysis/Normed/Affine/AsymptoticCone.lean,Mathlib/Order/Filter/Map.lean |
3 |
44 |
['AntoineChambert-Loir', 'YaelDillies', 'gasparattila', 'github-actions', 'mathlib4-dependent-issues-bot'] |
YaelDillies assignee:YaelDillies |
38-61467 1 month ago |
38-64752 1 month ago |
52-82289 52 days |
22043 |
YaelDillies author:YaelDillies |
chore: shortcut instance for `Neg ℤˣ` |
This lets us avoid importing `Ring` in downstream files (most of the effect is to come).
---
[](https://gitpod.io/from-referrer/)
|
file-removed
t-algebra
label:t-algebra$ |
20/47 |
Mathlib.lean,Mathlib/Algebra/GCDMonoid/Nat.lean,Mathlib/Algebra/Group/Int/Units.lean,Mathlib/Algebra/Order/Ring/Abs.lean,Mathlib/Algebra/Ring/Int/Units.lean,Mathlib/Algebra/Ring/NegOnePow.lean,Mathlib/Data/Fintype/Units.lean,Mathlib/Data/Int/AbsoluteValue.lean,Mathlib/Data/Int/Associated.lean,Mathlib/GroupTheory/HNNExtension.lean,Mathlib/NumberTheory/NumberField/Basic.lean,MathlibTest/Zify.lean |
12 |
16 |
['YaelDillies', 'eric-wieser', 'github-actions', 'j-loreaux', 'leanprover-community-bot-assistant', 'mathlib-bors'] |
erdOne assignee:erdOne |
38-34906 1 month ago |
121-76747 3 months ago |
206-49777 206 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'] |
kim-em assignee:kim-em |
38-34901 1 month ago |
81-66326 2 months ago |
85-35923 85 days |
26580 |
vasnesterov author:vasnesterov |
feat(Tactic/Order): translate linear orders to `Int` |
It was [pointed out](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/tactic.20for.20partial.20orders/near/515897754) that `order` is not complete for linear orders with lattice operations (while it remains complete for linear orders without lattice operations and for general lattices without assuming linearity). The problem for linear orders with lattice operations is NP-hard, but it can be translated from an arbitrary type to `Int` and then solved using a smart and efficient procedure (such as `omega`). This PR implements such a translation within the `order` tactic.
Co-authored-by: Aaron Liu
---
- [x] depends on: #26354
[](https://gitpod.io/from-referrer/) |
large-import
t-meta
|
302/22 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Order.lean,Mathlib/Tactic/Order/Graph/Basic.lean,Mathlib/Tactic/Order/Preprocessing.lean,Mathlib/Tactic/Order/ToInt.lean,MathlibTest/order.lean |
7 |
4 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'vasnesterov'] |
alexjbest assignee:alexjbest |
38-34900 1 month ago |
62-3189 2 months ago |
62-4886 62 days |
26679 |
robin-carlier author:robin-carlier |
feat(CategoryTheory/Limits/Shapes/Pullback/Categorical): 2-functoriality of `CatCommSqOver` |
This PR uses the notion of categorical cospan transforms from #26412 and its bicategory-like notations from #26447 to provide API for 2-functoriality of the construction `CatCommSqOver F G X`. We show that `ψ : CatCospanTransform F G F' G'` defines a functor `CatCommSqOver F G X ⥤ CatCommSqOver F' G' X`, and that a functor `U : X ⥤ Y` induces a functor `CatCommSqOver F G Y ⥤ CatCommSqOver F G X` via precomposition. We give the battery of lemma that shows that these constructions are components of a `Cat`-valued "bipseudofunctor", although we cannot state it this way to keep things unbundled and universe polymorphic.
---
- [x] depends on: #26447
I apologize in advance, for this one is very boring. As usual, the higher order lemmas are found by aesop_cat and are not marked simp, but I still want to state these explicitly so that in case automation goes wrong, "manual formal bicategory manipulations" remain an option.
A design choice was made here. Instead of stating this kind of functoriality for the categorical pullback itself, I chose to state everything in terms of `CatCommSqOver`, i.e in terms of the pseudofunctorial construction corepresented by the categorical pullback. The rationale here is that while we could have done everything only at the level of the categorical pullback itself, I believe this design will allow for easier manipulations of categorical pullback *squares*.
Actual bifunctoriality of the categorical pullback (and thus equivalence invariance, which is the key point of the notion compared to the strict pullback) will be in future PRs.
[](https://gitpod.io/from-referrer/)
|
t-category-theory |
364/1 |
Mathlib/CategoryTheory/Limits/Shapes/Pullback/Categorical/Basic.lean |
1 |
4 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'robin-carlier'] |
dagurtomas assignee:dagurtomas |
38-10624 1 month ago |
49-71335 1 month ago |
59-18574 59 days |
28032 |
grunweg author:grunweg |
feat: support Partial{Homeomorph,Equiv} in differential geometry elaborators |
---
[](https://gitpod.io/from-referrer/)
|
t-differential-geometry |
852/0 |
Mathlib.lean,Mathlib/Geometry/Manifold/Elaborators.lean,Mathlib/Geometry/Manifold/Traces.lean,MathlibTest/DifferentialGeometry/Elaborators.lean,scripts/noshake.json |
5 |
1 |
['github-actions'] |
nobody |
38-2526 1 month ago |
38-2526 1 month ago |
38-2591 38 days |
28026 |
kim-em author:kim-em |
feat: grind annotations for `Disjoint` |
---
[](https://gitpod.io/from-referrer/)
|
|
89/46 |
Archive/Imo/Imo2001Q3.lean,Mathlib/Data/Set/Disjoint.lean,Mathlib/Order/BoundedOrder/Basic.lean,Mathlib/Order/BoundedOrder/Lattice.lean,Mathlib/Order/Disjoint.lean,Mathlib/Order/Lattice.lean |
6 |
4 |
['github-actions', 'grunweg', 'leanprover-bot'] |
nobody |
37-86240 1 month ago |
38-18559 1 month ago |
0-0 0 seconds |
23669 |
erdOne author:erdOne |
feat(FieldTheory): abelian extensions |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
delegated
label:t-algebra$ |
74/0 |
Mathlib.lean,Mathlib/FieldTheory/Galois/Abelian.lean,Mathlib/NumberTheory/Cyclotomic/Gal.lean |
3 |
16 |
['acmepjz', 'alreadydone', 'chrisflav', 'erdOne', 'github-actions', 'mathlib-bors', 'riccardobrasca', 'xroblot'] |
riccardobrasca assignee:riccardobrasca |
37-77945 1 month ago |
66-82185 2 months ago |
29-68817 29 days |
26770 |
Jun2M author:Jun2M |
feat(Combinatorics/Graph) : subgraph relations and operations on `Graph` |
This PR creates a new file `Combinatorics/Graph/Subgraph.lean`. In it, the PR introduces a partial order on graphs by subgraph relation, defines relations `IsInducedSubgraph`, `IsSpanningSubgraph` and `IsClosedSubgraph`. Further, it introduce operations `EdgeRestrict`, `EdgeDelete`, `induce` and `VertexDelete`.
Co-authored-by: Peter Nelson
---
[](https://gitpod.io/from-referrer/)
|
t-combinatorics |
703/0 |
Mathlib.lean,Mathlib/Combinatorics/Graph/Subgraph.lean |
2 |
1 |
['github-actions'] |
awainverse assignee:awainverse |
37-34905 1 month ago |
70-46383 2 months ago |
70-46424 70 days |
28074 |
grunweg author:grunweg |
Isbilinearmap |
TODO see if it builds, move everything to the right place, add docs.
update Pr description - written by Patrick, part of #26221 (and prereq for #28056)
---
[](https://gitpod.io/from-referrer/)
|
WIP |
64/0 |
Mathlib/Analysis/Normed/Module/FiniteDimension.lean,Mathlib/LinearAlgebra/BilinearMap.lean |
2 |
1 |
['github-actions'] |
nobody |
37-5891 1 month ago |
37-8283 1 month ago |
0-2 2 seconds |
27229 |
WilliamCoram author:WilliamCoram |
feat(GroupTheory/DoubleCoset): multiple lemmas |
From FLT
---
[](https://gitpod.io/from-referrer/)
|
t-group-theory
new-contributor
|
106/0 |
Mathlib/GroupTheory/DoubleCoset.lean |
1 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
mariainesdff assignee:mariainesdff |
36-78776 1 month ago |
36-79509 1 month ago |
53-41071 53 days |
27991 |
sinianluoye author:sinianluoye |
feat (Rat): add Rat.den_eq_of_add_den_eq_one and its dependent lemmas |
```lean4
example {q r : ℚ} (h : (q + r).den = 1) : q.den = r.den := by
```
It is so simple, but I couldn't find it in current mathlib repo.
---
[](https://gitpod.io/from-referrer/)
|
t-data
new-contributor
|
28/0 |
Mathlib/Data/Rat/Lemmas.lean |
1 |
14 |
['github-actions', 'sinianluoye', 'themathqueen'] |
nobody |
36-61491 1 month ago |
38-34494 1 month ago |
38-62545 38 days |
26765 |
KiringYJ author:KiringYJ |
feat(MeasureTheory/PiSystem): add π-λ theorem and SetLike instance |
Add two small features to `MeasureTheory/PiSystem`:
1. SetLike instance
`instance : SetLike (DynkinSystem α) (Set α)`
This lets us write `s ⊆ d` and `t ∈ d` for a DynkinSystem `d`, matching usual mathlib style.
2. `DynkinSystem.pi_lambda` lemma
Classical π‑λ theorem: if a π‑system `s` is contained in a Dynkin system `d`, every set measurable for `σ(s)` is also in `d`.
Currently, mathlib exposes this result only indirectly (e.g. via `generateFrom_eq`). Although logically equivalent, it is not obvious at first glance that those lemmas are the π‑λ theorem. The new lemma states the result in its familiar textbook form, so users can recognise and cite it immediately.
Both pieces are under 10 lines, term‑mode only, and do not modify existing APIs.
No breaking changes.
No dependencies.
|
new-contributor
t-measure-probability
|
13/0 |
Mathlib/MeasureTheory/PiSystem.lean |
1 |
13 |
['EtienneC30', 'KiringYJ', 'github-actions', 'ocfnash'] |
RemyDegenne assignee:RemyDegenne |
36-34904 1 month ago |
43-70953 1 month ago |
70-58794 70 days |
27534 |
PierreQuinton author:PierreQuinton |
feat: a typeclass for `sSup`/`sInf` to be lawful |
Adds lawful infima and suprema type classes.
A preorder with lawful suprema: whenever a set has a least upper bound, `sSup` returns a least upper bound for that set.
A preorder with lawful infima: whenever a set has a greatest lower bound, `sInf` returns a greastest lower bound for that set.
---
[](https://gitpod.io/from-referrer/)
|
t-order |
121/8 |
Mathlib.lean,Mathlib/Order/CompleteLattice/Defs.lean,Mathlib/Order/LawfulSupInf.lean |
3 |
25 |
['PierreQuinton', 'YaelDillies', 'github-actions', 'plp127', 'vihdzp'] |
YaelDillies assignee:YaelDillies |
35-85081 1 month ago |
47-68378 1 month ago |
47-68410 47 days |
28111 |
euprunin author:euprunin |
chore: remove tactic `simp_lex` and use `simp` instead |
Motivation: `simp_lex` is just shorthand for `refine toLex.surjective.forall₃.2 ?_; rintro (a | a) (b | b) (c | c) <;> simp`, so plain `simp` seems preferable. |
t-data |
4/10 |
Mathlib/Data/Sum/Interval.lean |
1 |
5 |
['eric-wieser', 'euprunin', 'github-actions'] |
nobody |
35-72564 1 month ago |
35-72647 1 month ago |
35-80275 35 days |
28075 |
tristan-f-r author:tristan-f-r |
chore(Finsupp/Indicator): make non-classical |
This was surprising to see on a data-carrying definition.
---
[](https://gitpod.io/from-referrer/)
|
t-data
easy
awaiting-author
|
11/9 |
Mathlib/Algebra/BigOperators/Finsupp/Basic.lean,Mathlib/Data/Finsupp/Indicator.lean |
2 |
3 |
['github-actions', 'ocfnash', 'tristan-f-r'] |
nobody |
35-48540 1 month ago |
36-5959 1 month ago |
0-85904 23 hours |
25779 |
robin-carlier author:robin-carlier |
feat(CategoryTheory/Bicategory/NaturalTransformations): strong and lax natural transformations of lax functors |
Given two lax functors `F G` between bicategories, we define lax natural transformations as families of 1-morphisms `∀ a : B, F.obj a ⟶ G.obj a` equipped with a naturality 2-cell `∀ {a b : B} (f : a ⟶ b), app a ≫ G.map f ⟶ F.map f ≫ app b` that are required to satisfy conditions such as naturality, and compatibility with the `mapId` and `mapComp` fields of the source and target functors.
This notion dualizes the existing notion of oplax natural transformations between, and tries to narrow the current gap between lax and oplax functors in the library, where the latter has much more formalized API. For maintainability, The code tries to stay as aligned as possible with the code in `CategoryTheory.Bicategory.Naturaltransformations.Oplax`.
---
I followed the book by Johnson and Yau for the definition.
I made @yuma-mizuno and @callesonne authors of the files, as they are the authors of the original code for Oplax functors, which I basically copy-pasted and modified to make it work with lax functors. They should feel free to modify this if they want.
Next thing on the list is to tackle modifications between lax/strong natural transforms of lax transforms, as well as the category instance on lax functors.
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #25565.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/25565* |
t-category-theory |
286/0 |
Mathlib.lean,Mathlib/CategoryTheory/Bicategory/NaturalTransformation/Lax.lean,scripts/noshake.json |
3 |
3 |
['github-actions', 'yuma-mizuno'] |
joelriou assignee:joelriou |
35-34923 1 month ago |
70-10140 2 months ago |
91-54905 91 days |
27664 |
pechersky author:pechersky |
feat(Topology,Analysis): discrete topology metric space and normed groups |
Explicit construction of the discrete topology metric space and normed groups where `dist x y = 1` for all `x != y`
Provide PseudoMetricSpace, MetricSpace, Seminormed(Add)Group, and Normed(Add)Group constructions
---
[](https://gitpod.io/from-referrer/)
|
t-topology |
137/0 |
Mathlib/Analysis/Normed/Group/Basic.lean,Mathlib/Topology/MetricSpace/Basic.lean,Mathlib/Topology/MetricSpace/Pseudo/Constructions.lean |
3 |
3 |
['github-actions', 'kckennylau', 'pechersky'] |
urkud assignee:urkud |
35-34915 1 month ago |
45-24927 1 month ago |
45-24918 45 days |
26667 |
mariainesdff author:mariainesdff |
feat(FieldTheory/SplittingField/IsSplittingField): add IsScalarTower.splits, IsScalarTower.isAlgebraic |
Co-authored-by: @faenuccio
---
- [ ] depends on: #26666
[](https://gitpod.io/from-referrer/)
|
t-algebra
awaiting-author
label:t-algebra$ |
13/0 |
Mathlib/FieldTheory/SplittingField/IsSplittingField.lean |
1 |
7 |
['github-actions', 'mariainesdff', 'mathlib4-dependent-issues-bot', 'tb65536'] |
chrisflav assignee:chrisflav |
34-68069 1 month ago |
34-68069 1 month ago |
25-6784 25 days |
27525 |
Hagb author:Hagb |
(WIP) feat(Tactic/Linter/Indentation): add a linter for general indentation |
---
todo:
- [x] check whether some (direct or indirect) children of some kinds of parents are intended _strictly_ deeper than this parent.
For example:
```lean
example : Nat :=
Nat.add
1 -- should be strictly deeper than `Nat.add`?
2
```
- [ ] check whether some (direct or indirect) children of some kinds of parents are intended exactly N spaces deeper than this parent.
For example:
```lean
example : True :=
trivial -- should be exact 2 spaces deeper than 0 space of `example`
```
- [ ] some special cases, such as `calc`. https://github.com/leanprover-community/mathlib4/blob/5ebccb65951c70539ba1c36e53e079ac28b3fd23/Mathlib/Geometry/Manifold/Riemannian/Basic.lean#L452-L454
- [ ] add test cases
[](https://gitpod.io/from-referrer/)
|
large-import
t-linter
WIP
|
1364/1 |
Mathlib/Init.lean,Mathlib/Tactic/Linter/Indentation.lean,Mathlib/Tactic/Linter/Indentation/Basic.lean,Mathlib/Tactic/Linter/Indentation/Defs.lean,Mathlib/Tactic/Linter/Indentation/Linters.lean,MathlibTest/IndentationLinter.lean,lakefile.lean |
7 |
13 |
['Hagb', 'github-actions', 'grunweg'] |
nobody |
34-51242 1 month ago |
39-51499 1 month ago |
0-0 0 seconds |
28168 |
astrainfinita author:astrainfinita |
feat: hensel's lemma for topological rings |
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
t-algebra
t-topology
WIP
label:t-algebra$ |
616/0 |
Mathlib/RingTheory/Polynomial/Hensel.lean |
1 |
1 |
['github-actions'] |
nobody |
34-33975 1 month ago |
34-33985 1 month ago |
0-0 0 seconds |
23758 |
erdOne author:erdOne |
feat(Topology/Algebra): linearly topologized iff non-archimedean |
...for topological modules over compact rings or `ℤ`-finite rings
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebra
t-topology
awaiting-author
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 |
34-21773 1 month ago |
34-21773 1 month ago |
124-78308 124 days |
28119 |
JasperMS author:JasperMS |
feat(Data/Set/Pairwise): prove pairwise results for Chains, move `Set.pairwise_iUnion₂` |
Initiate a new file `Data/Set/Pairwise/Chain.lean` which makes some `Pairwise` results available to the `IsChain` predicate.
In the process, move `Set.pairwise_iUnion₂` to group it with similar results. Perform some variable harmonization.
Part of Carleson, original result by Edward van de Meent.
Moves:
- Set.pairwise_iUnion₂: from Data.Set.Lattice to Data.Set.Pairwise.Lattice
---
This PR was discussed and advice was given in [#mathlib4 > Novice questions on style and structure](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Novice.20questions.20on.20style.20and.20structure/with/533462814). Many thanks to those who helped me out!
Mathlib PRs are still new to me, so please point out where I can improve!
[](https://gitpod.io/from-referrer/)
|
carleson
t-data
new-contributor
|
56/12 |
Mathlib.lean,Mathlib/Data/Set/Lattice.lean,Mathlib/Data/Set/Pairwise/Chain.lean,Mathlib/Data/Set/Pairwise/Lattice.lean |
4 |
11 |
['JasperMS', 'Ruben-VandeVelde', 'edegeltje', 'github-actions'] |
nobody |
33-19413 1 month ago |
35-74109 1 month ago |
35-74549 35 days |
26901 |
5hv5hvnk author:5hv5hvnk |
feat: a simproc version of `compute_degree` |
Wrap `compute_degree` in a simproc for use by simp.
Closes #22219.
--- |
new-contributor
awaiting-CI
t-meta
awaiting-author
|
198/0 |
Mathlib.lean,Mathlib/Tactic/Simproc/PolynomialDegree.lean,MathlibTest/polynomial_degree_simproc.lean |
3 |
18 |
['5hv5hvnk', 'YaelDillies', 'adomani', 'github-actions'] |
nobody |
32-83868 1 month ago |
32-83868 1 month ago |
2-71043 2 days |
27850 |
fyqing author:fyqing |
feat: 0-dimensional manifolds are discrete and countable |
This is the converse direction of the classification of 0-dimensional manifolds. The other direction was shown in #22105.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-differential-geometry
awaiting-author
|
80/0 |
Mathlib.lean,Mathlib/Geometry/Manifold/ZeroDim.lean |
2 |
13 |
['fyqing', 'github-actions', 'grunweg', 'tb65536'] |
grunweg assignee:grunweg |
32-81476 1 month ago |
42-42292 1 month ago |
0-6418 1 hour |
28077 |
ShreckYe author:ShreckYe |
feat(Data/Finset/Card): add some more Pigeonhole Principle theorems `exists_ne_map_eq_of_card_image_lt` and `not_injOn_of_card_image_lt` |
`exists_ne_map_eq_of_card_image_lt` is a special case of `exists_ne_map_eq_of_card_lt_of_maps_to` where `t` is `s.image f`, and `not_injOn_of_card_image_lt` is its variant using `Set.InjOn`. I ran into some cases where such theorems would save me some time. |
t-data
new-contributor
|
10/0 |
Mathlib/Data/Finset/Card.lean |
1 |
4 |
['ShreckYe', 'github-actions', 'themathqueen'] |
nobody |
32-75602 1 month ago |
37-984 1 month ago |
37-1029 37 days |
27444 |
grunweg author:grunweg |
feat: generalise more lemmas to enorms |
The selection of lemmas may seem eclectic, but follows a clear path: I'm working on generalising the last section of `IntegrableOn.lean` to enorms. (This will be continued in a later PR.)
---
Commits can be reviewed independently.
- [x] depends on: #27419 (first commits)
- [x] depends on: #27456 (last commits)
[](https://gitpod.io/from-referrer/)
|
carleson
WIP
|
10/0 |
Mathlib/MeasureTheory/Function/L1Space/HasFiniteIntegral.lean |
1 |
3 |
['github-actions', 'grunweg', 'mathlib4-dependent-issues-bot'] |
nobody |
32-67036 1 month ago |
32-67072 1 month ago |
0-1886 31 minutes |
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
awaiting-author
|
261/0 |
Mathlib.lean,Mathlib/Topology/MetricSpace/CoveringNumbers.lean |
2 |
9 |
['ADedecker', 'RemyDegenne', 'YaelDillies', 'github-actions', 'j-loreaux'] |
j-loreaux assignee:j-loreaux |
32-65348 1 month ago |
35-52154 1 month ago |
45-38108 45 days |
28260 |
euprunin author:euprunin |
chore(Analysis/Fourier): golf entire `fourier_zero` and `fourier_zero'` using `simp` |
---
Show trace profiling of fourier_zero
### Trace profiling of `fourier_zero` before PR 28260
```diff
diff --git a/Mathlib/Analysis/Fourier/AddCircle.lean b/Mathlib/Analysis/Fourier/AddCircle.lean
index 6238f58476..99dbb05621 100644
--- a/Mathlib/Analysis/Fourier/AddCircle.lean
+++ b/Mathlib/Analysis/Fourier/AddCircle.lean
@@ -126,2 +126,3 @@ theorem fourier_coe_apply' {n : ℤ} {x : ℝ} :
-- simp normal form is `fourier_zero'`
+set_option trace.profiler true in
theorem fourier_zero {x : AddCircle T} : fourier 0 x = 1 := by
```
```
ℹ [2482/2482] Built Mathlib.Analysis.Fourier.AddCircle
info: Mathlib/Analysis/Fourier/AddCircle.lean:128:0: [Elab.async] [0.066690] elaborating proof of fourier_zero
[Elab.definition.value] [0.066228] fourier_zero
[Elab.step] [0.065930]
induction x using QuotientAddGroup.induction_on
simp only [fourier_coe_apply]
norm_num
[Elab.step] [0.065922]
induction x using QuotientAddGroup.induction_on
simp only [fourier_coe_apply]
norm_num
[Elab.step] [0.055636] simp only [fourier_coe_apply]
Build completed successfully.
```
### Trace profiling of `fourier_zero` after PR 28260
```diff
diff --git a/Mathlib/Analysis/Fourier/AddCircle.lean b/Mathlib/Analysis/Fourier/AddCircle.lean
index 6238f58476..0542519008 100644
--- a/Mathlib/Analysis/Fourier/AddCircle.lean
+++ b/Mathlib/Analysis/Fourier/AddCircle.lean
@@ -126,10 +126,8 @@ theorem fourier_coe_apply' {n : ℤ} {x : ℝ} :
-- simp normal form is `fourier_zero'`
+set_option trace.profiler true in
theorem fourier_zero {x : AddCircle T} : fourier 0 x = 1 := by
- induction x using QuotientAddGroup.induction_on
- simp only [fourier_coe_apply]
- norm_num
+ simp
-theorem fourier_zero' {x : AddCircle T} : @toCircle T 0 = (1 : ℂ) := by
- have : fourier 0 x = @toCircle T 0 := by rw [fourier_apply, zero_smul]
- rw [← this]; exact fourier_zero
+theorem fourier_zero' : @toCircle T 0 = (1 : ℂ) := by
+ simp
```
```
ℹ [2482/2482] Built Mathlib.Analysis.Fourier.AddCircle
info: Mathlib/Analysis/Fourier/AddCircle.lean:128:0: [Elab.async] [0.041217] elaborating proof of fourier_zero
[Elab.definition.value] [0.040843] fourier_zero
[Elab.step] [0.040316] simp
[Elab.step] [0.040305] simp
[Elab.step] [0.040291] simp
[Meta.isDefEq] [0.013042] ✅️ 0 • ?m =?= 0 • x
[Meta.isDefEq] [0.010734] ✅️ instHSMul =?= instHSMul
[Meta.isDefEq.delta] [0.010705] ✅️ instHSMul =?= instHSMul
[Meta.synthInstance] [0.010613] ✅️ SMulWithZero ℤ (AddCircle T)
[Meta.synthInstance] [0.010175] ✅️ apply @AddGroup.intSMulWithZero to SMulWithZero ℤ (AddCircle T)
[Meta.synthInstance.tryResolve] [0.010141] ✅️ SMulWithZero ℤ
(AddCircle T) ≟ SMulWithZero ℤ (AddCircle T)
[Meta.isDefEq] [0.010882] ❌️ ↑1 =?= ↑1
Build completed successfully.
```
---
Show trace profiling of fourier_zero'
### Trace profiling of `fourier_zero'` before PR 28260
```diff
diff --git a/Mathlib/Analysis/Fourier/AddCircle.lean b/Mathlib/Analysis/Fourier/AddCircle.lean
index 6238f58476..c97c6382dd 100644
--- a/Mathlib/Analysis/Fourier/AddCircle.lean
+++ b/Mathlib/Analysis/Fourier/AddCircle.lean
@@ -131,2 +131,3 @@ theorem fourier_zero {x : AddCircle T} : fourier 0 x = 1 := by
+set_option trace.profiler true in
theorem fourier_zero' {x : AddCircle T} : @toCircle T 0 = (1 : ℂ) := by
```
```
ℹ [2482/2482] Built Mathlib.Analysis.Fourier.AddCircle
info: Mathlib/Analysis/Fourier/AddCircle.lean:133:0: [Elab.command] [0.040228] theorem fourier_zero' {x : AddCircle T} : @toCircle T 0 = (1 : ℂ) :=
by
have : fourier 0 x = @toCircle T 0 := by rw [fourier_apply, zero_smul]
rw [← this]; exact fourier_zero
[Elab.definition.header] [0.039678] fourier_zero'
[Elab.step] [0.039292] expected type: Sort ?u.10460, term
@toCircle T 0 = (1 : ℂ)
[Elab.step] [0.039281] expected type: Sort ?u.10460, term
binrel% Eq✝ (@toCircle T 0) (1 : ℂ)
[Meta.synthInstance] [0.023079] ❌️ CoeT ℂ x Circle
info: Mathlib/Analysis/Fourier/AddCircle.lean:133:0: [Elab.async] [0.050645] elaborating proof of fourier_zero'
[Elab.definition.value] [0.049639] fourier_zero'
[Elab.step] [0.049079]
have : fourier 0 x = @toCircle T 0 := by rw [fourier_apply, zero_smul]
rw [← this]; exact fourier_zero
[Elab.step] [0.049067]
have : fourier 0 x = @toCircle T 0 := by rw [fourier_apply, zero_smul]
rw [← this]; exact fourier_zero
[Elab.step] [0.047714] have : fourier 0 x = @toCircle T 0 := by rw [fourier_apply, zero_smul]
[Elab.step] [0.047690] focus
refine
no_implicit_lambda%
(have : fourier 0 x = @toCircle T 0 := ?body✝;
?_)
case body✝ => with_annotate_state"by" (rw [fourier_apply, zero_smul])
[Elab.step] [0.047680]
refine
no_implicit_lambda%
(have : fourier 0 x = @toCircle T 0 := ?body✝;
?_)
case body✝ => with_annotate_state"by" (rw [fourier_apply, zero_smul])
[Elab.step] [0.047675]
refine
no_implicit_lambda%
(have : fourier 0 x = @toCircle T 0 := ?body✝;
?_)
case body✝ => with_annotate_state"by" (rw [fourier_apply, zero_smul])
[Elab.step] [0.016566] refine
no_implicit_lambda%
(have : fourier 0 x = @toCircle T 0 := ?body✝;
?_)
[Elab.step] [0.016520] expected type: ↑(toCircle 0) = 1, term
no_implicit_lambda%
(have : fourier 0 x = @toCircle T 0 := ?body✝;
?_)
[Elab.step] [0.016512] expected type: ↑(toCircle 0) = 1, term
(have : fourier 0 x = @toCircle T 0 := ?body✝;
?_)
[Elab.step] [0.016502] expected type: ↑(toCircle 0) = 1, term
have : fourier 0 x = @toCircle T 0 := ?body✝;
?_
[Elab.step] [0.016409] expected type: Sort ?u.12245, term
fourier 0 x = @toCircle T 0
[Elab.step] [0.016398] expected type: Sort ?u.12245, term
binrel% Eq✝ (fourier 0 x) (@toCircle T 0)
[Elab.step] [0.031091] case body✝ => with_annotate_state"by" (rw [fourier_apply, zero_smul])
[Elab.step] [0.031024] with_annotate_state"by" (rw [fourier_apply, zero_smul])
[Elab.step] [0.031018] with_annotate_state"by" (rw [fourier_apply, zero_smul])
[Elab.step] [0.031012] with_annotate_state"by" (rw [fourier_apply, zero_smul])
[Elab.step] [0.031006] (rw [fourier_apply, zero_smul])
[Elab.step] [0.031000] rw [fourier_apply, zero_smul]
[Elab.step] [0.030995] rw [fourier_apply, zero_smul]
[Elab.step] [0.030987] rw [fourier_apply, zero_smul]
[Elab.step] [0.030977] (rewrite [fourier_apply, zero_smul];
with_annotate_state"]" (try (with_reducible rfl)))
[Elab.step] [0.030972] rewrite [fourier_apply, zero_smul];
with_annotate_state"]" (try (with_reducible rfl))
[Elab.step] [0.030964] rewrite [fourier_apply, zero_smul];
with_annotate_state"]" (try (with_reducible rfl))
[Elab.step] [0.026599] rewrite [fourier_apply, zero_smul]
[Meta.isDefEq] [0.016855] ✅️ 0 • x =?= 0 • ?m
[Meta.isDefEq] [0.015512] ✅️ instHSMul =?= instHSMul
[Meta.isDefEq.delta] [0.015494] ✅️ instHSMul =?= instHSMul
[Meta.synthInstance] [0.015404] ✅️ SMulWithZero ℤ (AddCircle T)
[Meta.synthInstance] [0.014948] ✅️ apply @AddGroup.intSMulWithZero to SMulWithZero
ℤ (AddCircle T)
[Meta.synthInstance.tryResolve] [0.014922] ✅️ SMulWithZero ℤ
(AddCircle T) ≟ SMulWithZero ℤ (AddCircle T)
[Meta.isDefEq] [0.014466] ✅️ SMulWithZero ℤ
(AddCircle T) =?= SMulWithZero ℤ ?m.13159
[Meta.synthInstance] [0.010847] ✅️ Zero (AddCircle T)
Build completed successfully.
```
### Trace profiling of `fourier_zero'` after PR 28260
```diff
diff --git a/Mathlib/Analysis/Fourier/AddCircle.lean b/Mathlib/Analysis/Fourier/AddCircle.lean
index 6238f58476..f13a398896 100644
--- a/Mathlib/Analysis/Fourier/AddCircle.lean
+++ b/Mathlib/Analysis/Fourier/AddCircle.lean
@@ -127,9 +127,7 @@ theorem fourier_coe_apply' {n : ℤ} {x : ℝ} :
theorem fourier_zero {x : AddCircle T} : fourier 0 x = 1 := by
- induction x using QuotientAddGroup.induction_on
- simp only [fourier_coe_apply]
- norm_num
+ simp
-theorem fourier_zero' {x : AddCircle T} : @toCircle T 0 = (1 : ℂ) := by
- have : fourier 0 x = @toCircle T 0 := by rw [fourier_apply, zero_smul]
- rw [← this]; exact fourier_zero
+set_option trace.profiler true in
+theorem fourier_zero' : @toCircle T 0 = (1 : ℂ) := by
+ simp
```
```
ℹ [2482/2482] Built Mathlib.Analysis.Fourier.AddCircle
info: Mathlib/Analysis/Fourier/AddCircle.lean:131:0: [Elab.command] [0.045555] theorem fourier_zero' : @toCircle T 0 = (1 : ℂ) := by simp
[Elab.definition.header] [0.044962] fourier_zero'
[Elab.step] [0.044931] expected type: Sort ?u.10311, term
@toCircle T 0 = (1 : ℂ)
[Elab.step] [0.044920] expected type: Sort ?u.10311, term
binrel% Eq✝ (@toCircle T 0) (1 : ℂ)
[Meta.synthInstance] [0.031268] ❌️ CoeT ℂ x Circle
info: Mathlib/Analysis/Fourier/AddCircle.lean:131:0: [Elab.async] [0.027859] elaborating proof of fourier_zero'
[Elab.definition.value] [0.027542] fourier_zero'
[Elab.step] [0.027179] simp
[Elab.step] [0.027169] simp
[Elab.step] [0.027156] simp
[Meta.isDefEq] [0.011252] ❌️ ↑1 =?= ↑1
[Meta.isDefEq.delta] [0.010804] ❌️ ↑1 =?= ↑1
[Meta.isDefEq] [0.010774] ❌️ 1 =?= 1
[Meta.isDefEq] [0.010717] ❌️ { x // 0 ≤ x } =?= Circle
[Meta.isDefEq] [0.010706] ❌️ { x // 0 ≤ x } =?= ↥(Submonoid.unitSphere ℂ)
[Meta.isDefEq] [0.010684] ❌️ fun x ↦ 0 ≤ x =?= fun x ↦ x ∈ Submonoid.unitSphere ℂ
[Meta.isDefEq] [0.010675] ❌️ 0 ≤ x =?= x ∈ Submonoid.unitSphere ℂ
Build completed successfully.
```
---
[](https://gitpod.io/from-referrer/)
|
t-analysis
delegated
|
3/6 |
Mathlib/Analysis/Fourier/AddCircle.lean |
1 |
4 |
['eric-wieser', 'euprunin', 'github-actions', 'mathlib-bors'] |
nobody |
32-38835 1 month ago |
32-38835 1 month ago |
0-15279 4 hours |
27708 |
vihdzp author:vihdzp |
feat: unions and intersections of ordinals are ordinals |
As well as a bonus result `IsTransitive.empty_mem`.
---
[](https://gitpod.io/from-referrer/)
|
t-set-theory
awaiting-author
|
58/16 |
Mathlib/SetTheory/ZFC/Basic.lean,Mathlib/SetTheory/ZFC/Ordinal.lean |
2 |
4 |
['alreadydone', 'b-mehta', 'github-actions', 'vihdzp'] |
alreadydone assignee:alreadydone |
32-34936 1 month ago |
32-34936 1 month ago |
12-2927 12 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'] |
urkud assignee:urkud |
32-34921 1 month ago |
95-22231 3 months ago |
110-54163 110 days |
26089 |
WilliamCoram author:WilliamCoram |
feat: restricted power series form a ring |
We define restricted power series over a normed ring R, and show they form a ring when R has the ultrametric property
This is an update of [#23338](https://github.com/leanprover-community/mathlib4/pull/23338) to meet new expectations of PRs from forks.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-algebra
t-number-theory
label:t-algebra$ |
182/0 |
Mathlib.lean,Mathlib/RingTheory/PowerSeries/Restricted.lean |
2 |
7 |
['CBirkbeck', 'WilliamCoram', 'github-actions'] |
riccardobrasca assignee:riccardobrasca |
32-34919 1 month ago |
57-72214 1 month ago |
76-61644 76 days |
26547 |
robin-carlier author:robin-carlier |
feat(CategoryTheory/Limits/Shapes/Pullback/Categorical/CatCospanTransform): more lemmas about isomorphisms of `CatCospanTransform` |
We construct ways to extract left, right or base components of ismorphisms of `CatCospanTransform`, as well as various `IsIso` instances, and lemmas allowing to compute the left, right or base component of the inverse of a `CatCospanTransformMorphism` that has an `IsIso` instance.
---
- [x] depends on: #26412
[](https://gitpod.io/from-referrer/)
|
t-category-theory |
70/0 |
Mathlib/CategoryTheory/Limits/Shapes/Pullback/Categorical/CatCospanTransform.lean |
1 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
TwoFX assignee:TwoFX |
32-34917 1 month ago |
70-4454 2 months ago |
70-7498 70 days |
27000 |
gasparattila author:gasparattila |
feat(Analysis/Normed/Group/Quotient): isometric versions of isomorphisms |
This PR adds an isometric version of the third isomorphism theorem for groups and modules.
---
[](https://gitpod.io/from-referrer/)
|
large-import
new-contributor
t-analysis
|
49/2 |
Mathlib/Analysis/Normed/Group/Quotient.lean |
1 |
1 |
['github-actions'] |
urkud assignee:urkud |
32-34916 1 month ago |
63-74043 2 months ago |
63-74092 63 days |
27815 |
BGuillemet author:BGuillemet |
feat(CategoryTheory/Limits/Shapes/Products): add limMapPi and sigmaMapColim |
Add the canonical morphism from a limit to the product over its objects. Prove that it is a monomorphism.
Dually, add the canonical morphism to a colimit from the coproduc of its objects and prove that it is an epimorphism.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-category-theory
|
44/0 |
Mathlib/CategoryTheory/Limits/Shapes/Products.lean |
1 |
1 |
['github-actions'] |
jcommelin assignee:jcommelin |
32-34911 1 month ago |
42-81013 1 month ago |
42-81036 42 days |
27226 |
xcloudyunx author:xcloudyunx |
feat(Combinatorics/SimpleGraph): Add Subgraph.inclusion_edge_apply_coe and inclusion_edgeSet_apply_coe |
This PR continues the work from #25248.
Original PR: https://github.com/leanprover-community/mathlib4/pull/25248 |
new-contributor
t-combinatorics
awaiting-author
|
14/0 |
Mathlib/Combinatorics/SimpleGraph/Subgraph.lean |
1 |
3 |
['b-mehta', 'github-actions', 'xcloudyunx'] |
b-mehta assignee:b-mehta |
32-22863 1 month ago |
32-36943 1 month ago |
25-83942 25 days |
25480 |
ocfnash author:ocfnash |
feat: define a concrete model of the `𝔤₂` root system |
This is a bit of an experiment to test API but it should also make it easier to prove some properties of `𝔤₂`.
---
- [x] depends on: #25477
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebra
WIP
label:t-algebra$ |
120/15 |
Mathlib/LinearAlgebra/RootSystem/Defs.lean,Mathlib/LinearAlgebra/RootSystem/Finite/G2.lean,Mathlib/LinearAlgebra/RootSystem/Reduced.lean |
3 |
8 |
['eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'ocfnash'] |
nobody |
31-84199 1 month ago |
31-84216 1 month ago |
0-1 1 second |
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-ring-theory |
27/0 |
Mathlib/RingTheory/Ideal/GoingDown.lean |
1 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
alreadydone assignee:alreadydone |
31-34911 1 month ago |
39-3631 1 month ago |
116-65806 116 days |
27552 |
Equilibris author:Equilibris |
refactor: make universe levels visible in typevec |
This will be needed to allow `M.corec` to be generic across universes
---
[](https://gitpod.io/from-referrer/)
|
t-data
new-contributor
easy
|
16/10 |
Mathlib/Data/TypeVec.lean |
1 |
9 |
['Equilibris', 'eric-wieser', 'github-actions', 'plp127'] |
nobody |
31-16058 1 month ago |
31-54877 1 month ago |
47-67394 47 days |
22925 |
ggranberry author:ggranberry |
feat(Mathlib/PlaceHolder/ToeplitzHausdorff): Toeplitz-Hausdorff |
---
[](https://gitpod.io/from-referrer/)
|
will-close-soon
new-contributor
t-analysis
awaiting-author
WIP
help-wanted
|
411/0 |
Mathlib/PlaceHolder/ToeplitzHausdorff.lean,Mathlib/PlaceHolder/ToeplitzHausdorff_v2.lean |
2 |
11 |
['faenuccio', 'ggranberry', 'github-actions'] |
faenuccio assignee:faenuccio |
30-85387 30 days ago |
30-85590 30 days ago |
4-24257 4 days |
27180 |
ADedecker author:ADedecker |
feat: quotient of a monoid with zero by a multiplicative congruence |
---
My motivation is getting a more conceptual construction of [ValuativeRel.ValueGroupWithZero](https://leanprover-community.github.io/mathlib4_docs/Mathlib/RingTheory/Valuation/ValuativeRel.html#ValuativeRel.ValueGroupWithZero), but I think this is of independent interest.
[](https://gitpod.io/from-referrer/)
|
t-algebra
delegated
label:t-algebra$ |
141/26 |
Mathlib.lean,Mathlib/Data/Quot.lean,Mathlib/Data/Setoid/Basic.lean,Mathlib/GroupTheory/Congruence/Defs.lean,Mathlib/GroupTheory/Congruence/GroupWithZero.lean |
5 |
31 |
['ADedecker', 'eric-wieser', 'github-actions', 'mathlib-bors', 'ocfnash'] |
ocfnash assignee:ocfnash |
30-78544 30 days ago |
31-5352 1 month ago |
28-12053 28 days |
27934 |
JasperMS author:JasperMS |
feat(Order): no basic lemmas and some SuccOrder `biUnion` lemmas |
Documents that not all possible interval inclusion lemmas will be added to `Basic.lean`.
Also proves some `biUnion` results about `SuccOrder`.
-------
See also [Zulip: #mathlib4 > New contributor: #27934 (Order/Interval)](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/New.20contributor.3A.20.2327934.20.28Order.2FInterval.29).
This is my first attempt at a Mathlib PR, I have worked on the [Carleson project](https://github.com/fpvandoorn/carleson) so far. I have tried to find natural homes for these results, and worked to make them as general as possible.
Your feedback is welcome!
[](https://gitpod.io/from-referrer/)
|
carleson
new-contributor
t-order
|
40/10 |
Mathlib/Order/Interval/Set/Basic.lean,Mathlib/Order/SuccPred/Archimedean.lean,Mathlib/Order/SuccPred/IntervalSucc.lean |
3 |
10 |
['JasperMS', 'YaelDillies', 'github-actions'] |
YaelDillies assignee:YaelDillies |
30-54894 30 days ago |
32-9660 1 month ago |
40-9 40 days |
21031 |
YaelDillies author:YaelDillies |
chore: get rid of generic hom coercions |
---
[](https://gitpod.io/from-referrer/)
|
WIP |
161/166 |
Mathlib/Algebra/Group/Equiv/Basic.lean,Mathlib/Algebra/Group/Equiv/Defs.lean,Mathlib/Algebra/Group/Hom/Defs.lean,Mathlib/Algebra/Group/Subgroup/Map.lean,Mathlib/Algebra/Group/Units/Hom.lean,Mathlib/Algebra/GroupWithZero/Hom.lean,Mathlib/Algebra/Order/Hom/Monoid.lean,Mathlib/Algebra/Ring/Hom/Defs.lean,Mathlib/GroupTheory/MonoidLocalization/Basic.lean,Mathlib/Logic/Equiv/Defs.lean,Mathlib/Order/Hom/Basic.lean,Mathlib/Order/RelIso/Basic.lean,Mathlib/RingTheory/Valuation/Basic.lean |
13 |
13 |
['Vierkantor', 'YaelDillies', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-merge-conflict-bot', 'urkud'] |
nobody |
30-52455 30 days ago |
30-52517 30 days ago |
0-17 17 seconds |
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/4 |
Mathlib/Data/Nat/Basic.lean |
1 |
11 |
['b-mehta', 'eric-wieser', 'github-actions', 'leanprover-bot', 'mathlib4-merge-conflict-bot', 'mattrobball'] |
nobody |
30-39532 30 days ago |
30-39558 30 days ago |
81-44592 81 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'] |
eric-wieser assignee:eric-wieser |
30-34915 30 days ago |
124-23959 4 months ago |
147-48073 147 days |
27754 |
Parcly-Taxel author:Parcly-Taxel |
feat: `finCycle` as iterated `finRotate` |
Originally used in #25786, but eventually discovered to be unnecessary. |
t-logic |
26/5 |
Mathlib/Logic/Equiv/Fin/Rotate.lean |
1 |
1 |
['github-actions'] |
fpvandoorn assignee:fpvandoorn |
30-34907 30 days ago |
43-69663 1 month ago |
43-69714 43 days |
28057 |
plp127 author:plp127 |
feat(SuccOrder): simp lemma to refold `Order.succ` and `Order.pred` |
Adds `SuccOrder.succ_eq_succ` and `PredOrder.pred_eq_pred` to refold `SuccOrder.succ` and `PredOrder.pred` into `Order.succ` and `Order.pred`. These lemmas are marked `@[simp]`.
---
[](https://gitpod.io/from-referrer/)
|
t-order |
8/2 |
Mathlib/Order/SuccPred/Basic.lean |
1 |
3 |
['YaelDillies', 'github-actions', 'plp127', 'vihdzp'] |
bryangingechen assignee:bryangingechen |
29-79009 29 days ago |
37-60188 1 month ago |
37-60235 37 days |
27024 |
grunweg author:grunweg |
feat: Gram-Schmidt orthonormalisation for sections of a vector bundle |
Add a parametrised version of Gram-Schmidt, for sections of a topological vector bundle with a bundle metric.
This will be used to define orthonormal local frames.
From the path towards geodesics and the Levi-Civita connection.
Co-authored-by: Patrick Massot
---
- [x] depends on: #27023
[](https://gitpod.io/from-referrer/)
|
t-differential-geometry
awaiting-author
|
279/11 |
Mathlib.lean,Mathlib/Analysis/InnerProductSpace/GramSchmidtOrtho.lean,Mathlib/Topology/VectorBundle/GramSchmidtOrtho.lean,scripts/noshake.json |
4 |
70 |
['faenuccio', 'github-actions', 'grunweg', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'sgouezel'] |
sgouezel assignee:sgouezel |
29-62996 29 days ago |
29-62996 29 days ago |
28-73015 28 days |
27946 |
plp127 author:plp127 |
refactor: have `MetrizableSpace` not depend on `MetricSpace` |
Some theorems for uniform spaces with a countably generated uniformity do not mention their uniformity in any of the hypotheses or the conclusion (for example `UniformSpace.isCompact_iff_isSeqCompact`). This PR allows those theorems to be stated for (pseudo)metrizable spaces without importing the real numbers.
See also #2032
---
[](https://gitpod.io/from-referrer/)
|
t-topology |
129/102 |
Mathlib/Analysis/Fourier/RiemannLebesgueLemma.lean,Mathlib/Topology/Compactness/PseudometrizableLindelof.lean,Mathlib/Topology/GDelta/MetrizableSpace.lean,Mathlib/Topology/Metrizable/Basic.lean,Mathlib/Topology/Metrizable/ContinuousMap.lean,Mathlib/Topology/Metrizable/Real.lean,Mathlib/Topology/Metrizable/Uniformity.lean |
7 |
7 |
['github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot'] |
urkud assignee:urkud |
29-34892 29 days ago |
39-3177 1 month ago |
39-55055 39 days |
26125 |
faenuccio author:faenuccio |
first commit |
---
[](https://gitpod.io/from-referrer/)
|
dependency-bump
WIP
|
56/1 |
Hammer/experiment1.lean,lake-manifest.json,lakefile.lean |
3 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
29-7852 29 days ago |
29-7852 29 days ago |
0-19 19 seconds |
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$ |
60/76 |
Mathlib/RingTheory/RingHom/FinitePresentation.lean |
1 |
5 |
['chrisflav', 'erdOne', 'github-actions', 'mathlib4-dependent-issues-bot'] |
kim-em assignee:kim-em |
28-54593 28 days ago |
76-75676 2 months ago |
76-75720 76 days |
27974 |
smmercuri author:smmercuri |
feat: `Field`, `FiniteDimensional` and `Algebra.IsSeparable` instances for `WithAbs` |
This PR continues the work from #24870.
Original PR: https://github.com/leanprover-community/mathlib4/pull/24870 |
large-import
t-analysis
awaiting-author
|
14/1 |
Mathlib/Analysis/Normed/Field/WithAbs.lean |
1 |
2 |
['github-actions', 'j-loreaux'] |
j-loreaux assignee:j-loreaux |
28-20824 28 days ago |
28-20824 28 days ago |
10-66566 10 days |
28512 |
euprunin author:euprunin |
chore(Data/List): golf entire `getLast_append_of_right_ne_nil` and `finRange_map_getElem` |
---
[](https://gitpod.io/from-referrer/)
|
t-data |
4/9 |
Mathlib/Data/List/Basic.lean,Mathlib/Data/List/FinRange.lean |
2 |
1 |
['github-actions'] |
nobody |
28-2312 28 days ago |
28-2312 28 days ago |
28-2362 28 days |
27196 |
YaelDillies author:YaelDillies |
refactor(Polynomial/Bivariate): swap `X` and `Y` for improved notation |
This way, `X` keeps on being `X`.
From Toric
---
[](https://gitpod.io/from-referrer/)
|
toric
t-algebra
WIP
label:t-algebra$ |
3/3 |
Mathlib/Algebra/Polynomial/Bivariate.lean |
1 |
3 |
['YaelDillies', 'alreadydone', 'github-actions'] |
nobody |
27-79402 27 days ago |
43-13542 1 month ago |
15-75841 15 days |
26107 |
xroblot author:xroblot |
feat(NumberField/IsCM): first results about the action of `complexConjugation` on units |
Define the subgroup of real units of a CM field and prove that it is equal to the subgroup of units fixed by the complex conjugation.
---
- [x] depends on: #23536
- [x] depends on: #23453
- [x] depends on: #26746
|
t-number-theory |
170/8 |
Mathlib/GroupTheory/GroupAction/FixedPoints.lean,Mathlib/NumberTheory/NumberField/CMField.lean,Mathlib/NumberTheory/NumberField/Units/Basic.lean |
3 |
4 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'xroblot'] |
tb65536 assignee:tb65536 |
27-34900 27 days ago |
34-37768 1 month ago |
34-42528 34 days |
28141 |
YaelDillies author:YaelDillies |
chore: deprecate `BialgHom.coe_toLinearMap` |
`BialgHom.toLinearMap` is a fake projection.
From Toric
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
toric
easy
|
5/11 |
Mathlib/RingTheory/Bialgebra/Hom.lean |
1 |
8 |
['YaelDillies', 'eric-wieser', 'github-actions'] |
alreadydone assignee:alreadydone |
27-34895 27 days ago |
35-12024 1 month ago |
35-12020 35 days |
27105 |
xroblot author:xroblot |
feat(Ring/DedekindDomain): formula for the splitting of prime ideals in an extension |
This PR just puts together all the results that were already there to deduce:
```lean
map (algebraMap S R) p = ∏ P ∈ p.primesOver R, P ^ p.ramificationIdx (algebraMap S R) P
```
for `p` a maximal ideal of a ring `S` and `R` an extension of `S` that is a Dedekind ring.
Note. There is a significant import increase in the file `RingTheory.DedekindDomain.Factorization`. However, this file is almost a leaf file so this increase only affects a limited number of files. If the increase is too big, a new file, say `RingTheory.DedekindDomain.PrimeSplitting`, can be added instead.
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebra
t-number-theory
label:t-algebra$ |
88/2 |
Mathlib/RingTheory/DedekindDomain/Factorization.lean,Mathlib/RingTheory/DedekindDomain/Ideal/Basic.lean,Mathlib/RingTheory/DedekindDomain/Ideal/Lemmas.lean,Mathlib/RingTheory/Ideal/Operations.lean,Mathlib/RingTheory/Ideal/Over.lean |
5 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-merge-conflict-bot'] |
mariainesdff assignee:mariainesdff |
27-10132 27 days ago |
27-10149 27 days ago |
60-40397 60 days |
28527 |
grunweg author:grunweg |
feat: add ContMDiff.congr |
I wanted this lemma both while working on an early version of #28056 and while working on #23040: time to add it.
Besides, it fills a natural API gap.
---
[](https://gitpod.io/from-referrer/)
|
t-differential-geometry
easy
|
10/0 |
Mathlib/Geometry/Manifold/ContMDiff/Defs.lean |
1 |
3 |
['github-actions', 'grunweg', 'peabrainiac'] |
nobody |
26-79083 26 days ago |
27-59410 27 days ago |
27-59716 27 days |
26349 |
mans0954 author:mans0954 |
feat(Analysis/SpecialFunctions/Trigonometric/Basic): sin and cos of multiples of π / 3 |
This PR continues the work from #25009.
Original PR: https://github.com/leanprover-community/mathlib4/pull/25009 |
t-analysis
help-wanted
|
159/0 |
Mathlib/Algebra/Order/Monoid/NatCast.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Basic.lean,Mathlib/Data/Nat/Cast/Defs.lean,MathlibTest/trigonometry.lean |
4 |
3 |
['github-actions', 'mans0954', 'themathqueen'] |
nobody |
26-51014 26 days ago |
40-1899 1 month ago |
5-42837 5 days |
28497 |
euprunin author:euprunin |
chore: golf entire `nonneg_iff_isSelfAdjoint_and_spectrumRestricts`, `tail_append_singleton_of_ne_nil` and `isLocalHom_residue` |
---
[](https://gitpod.io/from-referrer/)
|
awaiting-author |
6/16 |
Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Instances.lean,Mathlib/Data/List/Basic.lean,Mathlib/RingTheory/LocalRing/ResidueField/Basic.lean |
3 |
2 |
['Ruben-VandeVelde', 'github-actions'] |
nobody |
26-49323 26 days ago |
26-49323 26 days ago |
1-84232 1 day |
28557 |
ShreckYe author:ShreckYe |
feat(Data/Nat/Factorization): some results on equality of powers of naturals proved from factorization |
I came across some math olympiad problems in number theory that could benefit from these theorems, expecially those on the prime power equality `p ^ m = a ^ n`. A specialized `eq_of_factorization_eq'` is added BTW to help with proof search. |
t-data |
102/0 |
Mathlib/Data/Nat/Factorization/Basic.lean,Mathlib/Data/Nat/Factorization/Defs.lean,Mathlib/Data/Nat/Factorization/PrimePow.lean |
3 |
1 |
['github-actions'] |
nobody |
26-46182 26 days ago |
26-63538 26 days ago |
26-63583 26 days |
28505 |
kim-em author:kim-em |
feat: linter for stale deprecated attrs |
- add a linter that reports `@[deprecated]` attributes with `since` dates more than three months old
- enable the linter by default via `Mathlib.Init`
Before merging we'll set back to 6 months, and disable by default.
- [ ] depends on: #28510
------
https://chatgpt.com/codex/tasks/task_e_68a00343bc148321a9528a8264d81536 |
large-import
t-linter
|
70/0 |
Mathlib/Init.lean,Mathlib/Tactic/Linter/DeprecatedAttr.lean |
2 |
6 |
['bryangingechen', 'github-actions', 'kim-em', 'mathlib4-dependent-issues-bot'] |
nobody |
26-36760 26 days ago |
27-40889 27 days ago |
0-0 0 seconds |
28198 |
Sebi-Kumar author:Sebi-Kumar |
feat(Analysis/InnerProductSpace/PiL2): Add instances for EuclideanSpace rank and EuclideanSpace being infinite |
Add an instance for `Fact (Module.finrank 𝕜 (EuclideanSpace 𝕜 (Fin n)) = n)` which is needed to apply [stereographic'](https://leanprover-community.github.io/mathlib4_docs/Mathlib/Geometry/Manifold/Instances/Sphere.html#stereographic') to EuclideanSpace. Also add an instance for `Infinite (EuclideanSpace 𝕜 ι)` where `ι` is a nonempty fintype. I wasn't sure if these should go in separate pull requests, but they seemed similar enough to me. Thank you to Kenny Lau for the suggestions at [#mathlib4 > Instances for EuclideanSpace](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Instances.20for.20EuclideanSpace).
---
To provide additional context, I am new to contributing to Mathlib, and I am doing so as a part of the Fields Undergraduate Summer Research Program at the University of Western Ontario under the supervision of Chris Kapulkin and Daniel Carranza. My goal is to contribute that the `n`-sphere is simply connected for `n > 1`.
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-analysis
|
6/0 |
Mathlib/Analysis/InnerProductSpace/PiL2.lean |
1 |
1 |
['github-actions'] |
urkud assignee:urkud |
26-34896 26 days ago |
33-48132 1 month ago |
33-48175 33 days |
28580 |
kmill author:kmill |
refactor: simplify implementation of `filter_upwards` |
This PR makes a few changes to `filter_upwards`:
- it uses `focus`, which prevents multiGoalLinter from ever blaming the tactics used inside its implementation
- it constructs the whole proof syntax and elaborates it at once using `evalTactic` and `refine`, rather than using the lower-level TermElab API, which can lose track of goals
- it's written in a way that doesn't require goals to be in some particular order
This was motivated by some multiGoalLinter issues I ran into when working on https://github.com/leanprover/lean4/pull/9942
---
[](https://gitpod.io/from-referrer/)
|
t-order
t-meta
|
14/16 |
Mathlib/Order/Filter/Defs.lean |
1 |
1 |
['github-actions'] |
nobody |
26-22424 26 days ago |
26-31297 26 days ago |
26-31279 26 days |
27302 |
tristan-f-r author:tristan-f-r |
feat(Fintype/Quotient): finLiftOn₂ |
The combination of [`Quotient.finLiftOn`](https://leanprover-community.github.io/mathlib4_docs/Mathlib/Data/Fintype/Quotient.html#Quotient.finLiftOn) and [`liftOn₂`](https://leanprover-community.github.io/mathlib4_docs/Init/Core.html#Quotient.liftOn%E2%82%82).
---
[](https://gitpod.io/from-referrer/)
|
t-data |
19/0 |
Mathlib/Data/Fintype/Quotient.lean |
1 |
10 |
['github-actions', 'kckennylau', 'tristan-f-r', 'vihdzp'] |
nobody |
26-19589 26 days ago |
55-31228 1 month ago |
55-31267 55 days |
5897 |
eric-wieser author:eric-wieser |
feat: add a `MonadError` instance for `ContT` |
We already have a `MonadExcept` instance; this promotes it to `MonadError`.
Note the issue with the existing `MonadExcept` instance still applies.
---
[](https://gitpod.io/from-referrer/)
|
t-meta
awaiting-author
|
16/0 |
Mathlib/Control/Monad/Cont.lean |
1 |
25 |
['Vierkantor', 'YaelDillies', 'eric-wieser', 'github-actions', 'kmill'] |
nobody |
25-84015 25 days ago |
422-18329 1 year ago |
339-53816 339 days |
28276 |
eric-wieser author:eric-wieser |
refactor: tidy `lift_unique` lemmas |
---
- [ ] depends on: #28275
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
37/20 |
Mathlib/Algebra/FreeAlgebra.lean,Mathlib/Algebra/Lie/UniversalEnveloping.lean,Mathlib/LinearAlgebra/DFinsupp.lean,Mathlib/LinearAlgebra/ExteriorAlgebra/Basic.lean |
4 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
25-83286 25 days ago |
25-83305 25 days ago |
0-0 0 seconds |
23881 |
YaelDillies author:YaelDillies |
feat: `ℝ≥0`-valued Lᵖ norm |
This is useful when inputting the Lp norm in places that expect a real number, like an exponent.
From LeanAPAP
---
[](https://gitpod.io/from-referrer/)
|
t-measure-probability
awaiting-author
|
218/6 |
Mathlib.lean,Mathlib/MeasureTheory/Function/LpSeminorm/Defs.lean,Mathlib/MeasureTheory/Function/LpSeminorm/NNLpNorm.lean,Mathlib/MeasureTheory/Function/LpSeminorm/TriangleInequality.lean |
4 |
20 |
['YaelDillies', 'b-mehta', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-merge-conflict-bot', 'sgouezel'] |
nobody |
25-73214 25 days ago |
25-73233 25 days ago |
13-15316 13 days |
28072 |
kckennylau author:kckennylau |
feat(RingTheory/Valuation): make tactic rw_val_equiv |
Co-authored by Aaron Liu and Bhavik Mehta.
A tactic to rewrite relations such as `max (v₁ x) (v₁ y) * v₁ z < 1` into `max (v₂ x) (v₂ y) * v₂ z < 1` , given `h : v₁.IsEquiv v₂`.
Allowed relations are `≤`, `<`, `=`, `≠`.
Allowed operations are: `0`, `1`, `v₁ r`, `⁻¹`, `^` (both `ℕ` and `ℤ`), `*`, `/`, `min`, `max`.
Examples:
```lean
example {R Γ₁ Γ₂ : Type} [Ring R]
[LinearOrderedCommMonoidWithZero Γ₁] [LinearOrderedCommMonoidWithZero Γ₂]
{v₁ : Valuation R Γ₁} {v₂ : Valuation R Γ₂}
(h : v₁.IsEquiv v₂) {y z : R} :
{x | v₁ x ^ 2 * min (v₁ y) (v₁ z) ≤ 1} = {x | v₂ x ^ 2 * min (v₂ y) (v₂ z) ≤ 1} := by
rw_val_equiv h
```
It is also possible to use `←` to rewrite in the opposite direction, and to use `at h1 h3 ⊢` to specify which hypotheses (and/or goal) to rewrite, similar to the syntax of `rw`. There is also `rwa_val_equiv` to work like `rwa`.
---
Zulip: [#Is there code for X? > Tactics for comparing equivalent valuations](https://leanprover.zulipchat.com/#narrow/channel/217875-Is-there-code-for-X.3F/topic/Tactics.20for.20comparing.20equivalent.20valuations)
[](https://gitpod.io/from-referrer/)
|
t-ring-theory |
455/13 |
Mathlib/RingTheory/Valuation/Basic.lean,MathlibTest/Simproc/ValEquiv.lean |
2 |
34 |
['b-mehta', 'eric-wieser', 'github-actions', 'kckennylau', 'pechersky', 'plp127'] |
erdOne assignee:erdOne |
25-34911 25 days ago |
35-56603 1 month ago |
36-31105 36 days |
28191 |
kckennylau author:kckennylau |
feat(Logic): tag Injective, Surjective, and Bijective with fun_prop |
---
Zulip:
* [#Is there code for X? > surjective is not funprop!](https://leanprover.zulipchat.com/#narrow/channel/217875-Is-there-code-for-X.3F/topic/surjective.20is.20not.20funprop!)
* [#mathlib4 > `fun_prop` for Injective/Surjective/Bijective?](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/.60fun_prop.60.20for.20Injective.2FSurjective.2FBijective.3F)
[](https://gitpod.io/from-referrer/)
|
t-meta |
16/0 |
Mathlib/Tactic/FunProp.lean |
1 |
3 |
['github-actions', 'grunweg', 'kckennylau'] |
alexjbest assignee:alexjbest |
25-34909 25 days ago |
32-71420 1 month ago |
33-49628 33 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
---
- [ ] depends on: #28367
- [ ] depends on: #28359
- [ ] depends on: #28368
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
awaiting-author
|
129/110 |
Mathlib/RingTheory/MatrixAlgebra.lean |
1 |
27 |
['Whysoserioushah', 'chrisflav', 'eric-wieser', 'github-actions', 'jcommelin', 'mathlib-bors', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'mattrobball'] |
chrisflav assignee:chrisflav |
25-8237 25 days ago |
25-8237 25 days ago |
63-50556 63 days |
28631 |
faenuccio author:faenuccio |
feat(Data\Nat\ModEq.lean): add grind attribute to ModEq |
---
[](https://gitpod.io/from-referrer/)
|
t-data
WIP
|
7/0 |
Mathlib/Data/Nat/ModEq.lean |
1 |
4 |
['faenuccio', 'github-actions', 'leanprover-bot'] |
nobody |
25-3268 25 days ago |
25-5787 25 days ago |
0-22 22 seconds |
26329 |
Timeroot author:Timeroot |
feat: Definition of `Clone` notations and typeclasses |
Definitions and notation typeclasses for #20051
---
This PR continues the work from #23459.
Original PR: https://github.com/leanprover-community/mathlib4/pull/23459
[](https://gitpod.io/from-referrer/) |
t-algebra
awaiting-CI
awaiting-author
label:t-algebra$ |
100/0 |
Mathlib.lean,Mathlib/Algebra/Clone/Defs.lean |
2 |
3 |
['Timeroot', 'YaelDillies', 'github-actions'] |
nobody |
25-1151 25 days ago |
25-1151 25 days ago |
0-21917 6 hours |
28581 |
bennett-chow author:bennett-chow |
fix: riemmanian -> riemannian |
changed riemmanian to riemannian
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-differential-geometry
awaiting-author
|
8/8 |
Mathlib/Geometry/Manifold/Riemannian/Basic.lean |
1 |
5 |
['bennett-chow', 'bryangingechen', 'github-actions', 'grunweg'] |
nobody |
24-83852 24 days ago |
25-72240 25 days ago |
0-40695 11 hours |
25070 |
erdOne author:erdOne |
feat(EllipticCurve): rational points on singular cuspidal cubics |
---
[](https://gitpod.io/from-referrer/)
|
t-algebraic-geometry
awaiting-author
|
123/0 |
Mathlib.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Singular/Cusp.lean |
2 |
11 |
['Multramate', 'acmepjz', 'adamtopaz', 'erdOne', 'github-actions', 'kckennylau'] |
adamtopaz assignee:adamtopaz |
24-63338 24 days ago |
24-63436 24 days ago |
90-52970 90 days |
27752 |
plp127 author:plp127 |
feat(Order): `NoBotOrder α` implies `NoMinOrder α` under `IsDirected α (· ≥ ·)` |
This PR continues the work from #24266.
Original PR: https://github.com/leanprover-community/mathlib4/pull/24266 |
t-order
awaiting-author
|
14/0 |
Mathlib/Order/Directed.lean |
1 |
4 |
['github-actions', 'j-loreaux', 'plp127'] |
nobody |
24-52527 24 days ago |
24-52527 24 days ago |
19-20394 19 days |
28125 |
nonisomorphiclinearmap author:nonisomorphiclinearmap |
feat(Combinatorics): basic definition of simplicial complexes |
This PR introduces the basic definition of a finite (abstract) simplicial complex, located in Mathlib/Combinatorics/SimplicialComplex/Basic.lean.
---
This is our first contribution to mathlib. This work was done as part of the Fields Institute Summer Undergraduate Program on formalization in topological combinatorics. Eventually, we aim to formalize Lovasz's proof of the Kneser Conjecture and this is a small stepping stone in that direction. Some other commits will shortly depend on this one.
We would like to acknowledge the Fields Institute for Research in Mathematical Sciences for their sponsorship. We would also like to thank our supervisors, Professor Chris Kapulkin and Mr. Daniel Carranza, for their guidance and support throughout this project. We would also like to thank our group members Tom Lindquist and Quang Minh Nguyen for our fruitful discussions. |
new-contributor
t-combinatorics
|
374/0 |
Mathlib.lean,Mathlib/Combinatorics/SimplicialComplex/Basic.lean,Mathlib/Combinatorics/SimplicialComplex/Category.lean,Mathlib/Combinatorics/SimplicialComplex/FacePoset.lean,Mathlib/Combinatorics/SimplicialComplex/Hom.lean |
5 |
1 |
['github-actions'] |
awainverse assignee:awainverse |
24-34919 24 days ago |
35-53388 1 month ago |
35-53430 35 days |
28153 |
kckennylau author:kckennylau |
feat(Simproc): Simproc for explicit diagonal matrices |
```lean
example : (diagonal ![37, -1] : Matrix (Fin 2) (Fin 2) ℤ) = !![37, 0; 0, -1] := by
simp
```
---
Shares code with #28148.
[](https://gitpod.io/from-referrer/)
|
t-meta |
114/0 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Simproc/Matrix.lean,scripts/noshake.json |
4 |
1 |
['github-actions'] |
alexjbest assignee:alexjbest |
24-34917 24 days ago |
34-59659 1 month ago |
34-59707 34 days |
28186 |
Sebi-Kumar author:Sebi-Kumar |
feat(Topology/Homotopy/Path): Add IsEquiv instance for Path.Homotopic |
Add `instance : IsEquiv (Path x₀ x₁) Homotopic` to the library. Allow use of lemmas like `of_eq` when proving two paths are homotopic.
---
To provide additional context, I am relatively new to contributing to Mathlib, and I am doing so as a part of the Fields Undergraduate Summer Research Program hosted at the University of Western Ontario and supervised by Chris Kapulkin and Daniel Carranza. My goal is to prove that the `n`-sphere is simply connected for `n > 1`.
Also, I am not super familiar with `IsEquiv` and when it should/shouldn't be used. I just wanted to use a lemma like `Path.Homotopic.of_eq` at one point while working on my code, and thought this was the best way to add such a result to the library.
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-topology
|
5/0 |
Mathlib/Topology/Homotopy/Path.lean |
1 |
4 |
['Sebi-Kumar', 'github-actions', 'kckennylau'] |
PatrickMassot assignee:PatrickMassot |
24-34916 24 days ago |
33-66246 1 month ago |
33-66291 33 days |
24514 |
b-mehta author:b-mehta |
chore(Int/GCD): use fuel in xgcd |
Modify the definition of xgcd to use fuel recursion, to allow it to be reduced in the kernel. As a consequence, this means the evaluation of field operations in ZMod p become provable by `rfl` and `decide`.
Zulip discussion: https://leanprover.zulipchat.com/#narrow/channel/270676-lean4/topic/opaque.20recursion.20definitions.20break.20mergeSort.20decidability
---
[](https://gitpod.io/from-referrer/)
|
t-data
awaiting-author
|
44/22 |
Mathlib/Data/Int/GCD.lean |
1 |
5 |
['astrainfinita', 'b-mehta', 'eric-wieser', 'github-actions', 'nomeata', 'urkud'] |
nobody |
24-8961 24 days ago |
76-38058 2 months ago |
58-34020 58 days |
26645 |
erdOne author:erdOne |
feat(RingTheory/PowerSeries): Construction of `Q` such that `P(Q(X)) = X` |
Co-authored-by: Junnosuke Koizumi
Co-authored-by: Hyeon, Seung-Hyeon
Co-authored-by: Yuichiro Taguchi
This contribution was created as part of the ZMC conference 2025 "Anabelian Geometry and its Computer Formalization".
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
awaiting-author
|
133/0 |
Mathlib/RingTheory/PowerSeries/Substitution.lean |
1 |
9 |
['chrisflav', 'erdOne', 'github-actions', 'kckennylau'] |
kbuzzard assignee:kbuzzard |
24-8791 24 days ago |
24-8791 24 days ago |
48-29860 48 days |
28680 |
vihdzp author:vihdzp |
feat: set has cardinality one iff singleton |
---
[](https://gitpod.io/from-referrer/)
|
t-set-theory
easy
awaiting-author
|
11/1 |
Mathlib/SetTheory/Cardinal/Basic.lean,Mathlib/SetTheory/Cardinal/Defs.lean |
2 |
5 |
['b-mehta', 'github-actions', 'kckennylau'] |
nobody |
23-75552 23 days ago |
23-75552 23 days ago |
0-24645 6 hours |
27443 |
yuanyi-350 author:yuanyi-350 |
Stacks tags |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
WIP
label:t-algebra$ |
6/3 |
Mathlib/Data/Nat/Init.lean,Mathlib/RingTheory/Localization/AtPrime/Basic.lean,Mathlib/RingTheory/Noetherian/Basic.lean |
3 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
23-70035 23 days ago |
28-71887 28 days ago |
0-990 16 minutes |
26300 |
igorkhavkine author:igorkhavkine |
feat(Analysis/Calculus/FDeriv): continuous differentiability from continuous partial derivatives on an open domain in a product space |
If a function `f : E × F → G` is continuously differentiable, then its partial derivatives along `E` and `F` are also continuous. The non-trivial converse implication holds when the partial derivatives are continuous on an open domain, and they can be added together to give the total derivative of `f`. See this [#mathlib4 > Partial derivatives @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Partial.20derivatives/near/520995477) and the containing thread for some discussion. The PR creates a new import (`Mathlib.Analysis.Calculus.FDeriv.Partial`), where other results about partial derivatives could go in the future.
---
*this is the migration of #25304 to the PR-from-fork workflow*
- [x] depends on: #25564
- [x] depends on: #26273
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-analysis
awaiting-author
WIP
|
497/0 |
Mathlib.lean,Mathlib/Analysis/Calculus/FDeriv/Partial.lean,Mathlib/Analysis/Normed/Module/Convex.lean,Mathlib/Analysis/Normed/Operator/BoundedLinearMaps.lean |
4 |
19 |
['YaelDillies', 'agjftucker', 'github-actions', 'igorkhavkine', 'mathlib4-dependent-issues-bot', 'sgouezel'] |
sgouezel assignee:sgouezel |
23-67097 23 days ago |
23-67097 23 days ago |
50-22679 50 days |
25795 |
dagurtomas author:dagurtomas |
chore(Condensed): introduce an abbrev for the equivalence of light condensed sets with a category of sheaves on a small site |
---
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #24522.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/24522* |
t-condensed |
39/0 |
Mathlib.lean,Mathlib/Condensed/Light/Small.lean |
2 |
1 |
['github-actions'] |
joneugster assignee:joneugster |
23-50032 23 days ago |
93-141 3 months ago |
93-121 93 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
- [x] depends on: #27239 |
t-topology
awaiting-author
|
424/0 |
Mathlib.lean,Mathlib/Topology/EMetricSpace/PairReduction.lean |
2 |
76 |
['DavidLedvinka', 'EtienneC30', 'RemyDegenne', 'github-actions', 'mathlib4-dependent-issues-bot', 'sgouezel'] |
nobody |
23-41670 23 days ago |
29-57394 29 days ago |
39-560 39 days |
26829 |
pechersky author:pechersky |
feat(RingTheory/Valuation): Valuation.leAddSubgroup and ideal/submodule versions of ltAddSubgroup |
Extracted from #25450 without changing how Valued works
---
[](https://gitpod.io/from-referrer/)
@faenuccio hopefully this bypasses any wait on #14752 because I am not changing Valued files. |
t-ring-theory |
172/0 |
Mathlib/RingTheory/Valuation/Basic.lean,Mathlib/RingTheory/Valuation/Integers.lean |
2 |
3 |
['JovanGerb', 'github-actions', 'mathlib4-merge-conflict-bot'] |
mariainesdff assignee:mariainesdff |
23-34928 23 days ago |
35-57251 1 month ago |
68-31768 68 days |
28352 |
agjftucker author:agjftucker |
feat(Analysis): add three little theorems relating argument to image |
These relate argument to image under a continuous function, given a Prop that eventually holds on a product of filters in domain and codomain. In fact the second pair of statements concern a segment whose end-points are the image. They should prove useful in PRs 26300 and 26985.
---
[](https://gitpod.io/from-referrer/)
|
t-analysis |
28/3 |
Mathlib/Analysis/Normed/Module/Convex.lean,Mathlib/Order/Filter/Prod.lean |
2 |
1 |
['github-actions'] |
sgouezel assignee:sgouezel |
23-34922 23 days ago |
30-59625 30 days ago |
30-66813 30 days |
26777 |
YaelDillies author:YaelDillies |
chore(Data/Set/Image): move `BooleanAlgebra` material to `Order` |
Eventually, all order properties should move out, but this is a good fourth step that will, among others, unblock #23177.
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-data
WIP
|
143/118 |
Mathlib/Algebra/Notation/Support.lean,Mathlib/Data/Set/Image.lean,Mathlib/Data/Set/Prod.lean,Mathlib/Data/Set/Restrict.lean,Mathlib/Data/Set/SymmDiff.lean,Mathlib/Logic/Equiv/Embedding.lean,Mathlib/Order/BooleanAlgebra/Set.lean,Mathlib/Order/CompleteBooleanAlgebra.lean |
8 |
8 |
['Ruben-VandeVelde', 'YaelDillies', 'github-actions', 'mathlib4-merge-conflict-bot'] |
bryangingechen assignee:bryangingechen |
23-7685 23 days ago |
23-7706 23 days ago |
2-29376 2 days |
26428 |
Ruben-VandeVelde author:Ruben-VandeVelde |
feat: norm_num support for Int.fract |
---
[](https://gitpod.io/from-referrer/)
|
t-data
t-meta
|
61/0 |
Mathlib/Data/Rat/Floor.lean,MathlibTest/norm_num_ext.lean |
2 |
6 |
['Rob23oba', 'github-actions', 'grunweg'] |
Rob23oba assignee:Rob23oba |
22-78032 22 days ago |
22-78032 22 days ago |
79-6116 79 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-ring-theory |
121/38 |
Mathlib/LinearAlgebra/BilinearForm/Properties.lean,Mathlib/RingTheory/DedekindDomain/Different.lean,Mathlib/RingTheory/Trace/Basic.lean |
3 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
adomani assignee:adomani |
22-76799 22 days ago |
22-76825 22 days ago |
78-44619 78 days |
26975 |
Whysoserioushah author:Whysoserioushah |
feat: a norm_num extension for complex numbers |
co-authored-by : @thefundamentaltheor3m, @hrmacbeth
---
[](https://gitpod.io/from-referrer/)
|
t-meta |
350/0 |
Mathlib.lean,Mathlib/Analysis/RCLike/Basic.lean,Mathlib/Tactic.lean,Mathlib/Tactic/NormNum/NormNumI.lean,MathlibTest/norm_numI.lean |
5 |
47 |
['Whysoserioushah', 'dupuisf', 'eric-wieser', 'github-actions', 'hrmacbeth'] |
robertylewis assignee:robertylewis |
22-74722 22 days ago |
57-59038 1 month ago |
57-63352 57 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
awaiting-author
|
44/0 |
Mathlib/AlgebraicGeometry/EllipticCurve/Affine/Point.lean |
1 |
12 |
['MichaelStollBayreuth', 'Multramate', 'acmepjz', 'dagurtomas', 'github-actions', 'kckennylau'] |
dagurtomas assignee:dagurtomas |
22-70076 22 days ago |
22-70076 22 days ago |
64-11252 64 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
t-logic
|
159/0 |
Mathlib/Data/Rel.lean,Mathlib/ModelTheory/Definability.lean,scripts/noshake.json |
3 |
15 |
['Timeroot', 'github-actions', 'staroperator'] |
fpvandoorn assignee:fpvandoorn |
22-41198 22 days ago |
40-1867 1 month ago |
81-27556 81 days |
28432 |
euprunin author:euprunin |
chore(CategoryTheory/Monoidal): golf entire `counitInv_app_comp_functor_map_η_inverse` |
---
[](https://gitpod.io/from-referrer/)
|
t-category-theory |
2/5 |
Mathlib/CategoryTheory/Monoidal/Functor.lean |
1 |
1 |
['github-actions'] |
adamtopaz assignee:adamtopaz |
22-34916 22 days ago |
29-54241 29 days ago |
29-54287 29 days |
27937 |
madvorak author:madvorak |
feat(Logic/Basic): `congr_heq₂` |
---
[](https://gitpod.io/from-referrer/)
|
t-logic
awaiting-author
|
6/0 |
Mathlib/Logic/Basic.lean |
1 |
8 |
['YaelDillies', 'github-actions', 'madvorak', 'vihdzp'] |
fpvandoorn assignee:fpvandoorn |
22-3780 22 days ago |
22-3787 22 days ago |
17-70200 17 days |
28718 |
imbrem author:imbrem |
Added chosen finite coproducts |
Added basic `ChosenFiniteCoproducts` class, and started porting some of the lemmas about `ChosenFiniteProducts` suitably translated
---
This, combined with #20182 modified to use chosen finite coproducts and premonoidal categories (#21488), should be enough for me to formalize strong Elgot categories, and hence a lot of categorical iteration theory for my PhD thesis.
Re-done from #21603 to deal with changes in #24399 and #24390
Eventually, if we really want to harmonize approaches, we could introduce an `AddMonoidalCategory` struct and do the analogous to #24399 and #24390 for additive monoidal structure, but that seems like a massive overcomplication for now. It would allow formalizing fun things like rig categories, though. |
new-contributor
t-category-theory
awaiting-author
|
290/0 |
Mathlib.lean,Mathlib/CategoryTheory/ChosenFiniteCoproducts.lean |
2 |
6 |
['YaelDillies', 'github-actions', 'imbrem', 'robin-carlier'] |
nobody |
21-80392 21 days ago |
23-18651 23 days ago |
0-24930 6 hours |
26870 |
grunweg author:grunweg |
feat: mdifferentiableOn_section_of_mem_baseSet₀ |
The `MDifferentiable` analogue of `contMDiffOn_section_of_mem_baseSet₀`.
From the path towards geodesics and the Levi-Civita connection.
Co-authored-by: Patrick Massot
---
- [x] depends on: #26866
[](https://gitpod.io/from-referrer/)
|
t-differential-geometry |
125/0 |
Mathlib/Geometry/Manifold/VectorBundle/MDifferentiable.lean |
1 |
4 |
['github-actions', 'grunweg', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
sgouezel assignee:sgouezel |
21-61212 21 days ago |
57-76695 1 month ago |
57-76853 57 days |
28422 |
euprunin author:euprunin |
chore(Data/Fin): deprecate `Fin.mul_one'` (duplicate) |
---
[](https://gitpod.io/from-referrer/)
|
t-data
awaiting-author
|
3/8 |
Mathlib/Data/Fin/Basic.lean,Mathlib/Data/ZMod/Defs.lean |
2 |
2 |
['eric-wieser', 'github-actions'] |
nobody |
21-47416 21 days ago |
21-47416 21 days ago |
8-10801 8 days |
26267 |
vasnesterov author:vasnesterov |
feat(Analysis/Calculus): Taylor series converges to function on whole ball |
* Prove `FormalMultilinearSeries.AnalyticOnNhd`: the sum of series is analytic on its ball of convergence.
* Prove `AnalyticOn.hasFPowerSeriesOnBall`: a variant of `AnalyticAt.hasFPowerSeriesAt` which gives convergence to the function on the ball of convergence.
---
- [x] depends on: #23745
- [x] depends on: #23747
- [x] depends on: #23748
- [x] depends on: #26247
This PR continues the work from #23749.
Original PR: https://github.com/leanprover-community/mathlib4/pull/23749 |
t-analysis |
65/0 |
Mathlib.lean,Mathlib/Analysis/Analytic/ChangeOrigin.lean,Mathlib/Analysis/Calculus/IteratedDeriv/ConvergenceOnBall.lean |
3 |
5 |
['github-actions', 'grunweg', 'mathlib4-dependent-issues-bot', 'vasnesterov'] |
urkud assignee:urkud |
21-46907 21 days ago |
23-72110 23 days ago |
70-56983 70 days |
28242 |
robin-carlier author:robin-carlier |
feat(CategoryTheory/Bicategory): EqToHom for bicategories |
We generalize the `eqToHom` construction from `Category` to `CategoryStruct`, allowing its usage in bicategorical contexts.
We introduce a file `CategoryTheory/Bicategory/EqToHom` that records some of the properties of `eqToHom`s 1-morphisms and 2-morphisms, such as the transitivity up to isomorphism of `eqToHom` 1-morphisms, and congruence lemmas for unitors, associators and whiskering with respects to `eqToHom` 2-morphisms.
This generalization and these congruence lemmas will be used to define icons between lax functors, and work with categories of strictly unitary lax/pseudo-functors (e.g for pseudocomposable arrows and lax-composable arrows in bicategories, which are part of the definitions of nerve constructions in bicategories).
---
A follow-up PR will move some existing `eqToHom`-related lemmas from `CategoryTheory/Bicategory/Strict` to this new file.
[](https://gitpod.io/from-referrer/)
|
t-category-theory |
150/4 |
Mathlib.lean,Mathlib/CategoryTheory/Bicategory/EqToHom.lean,Mathlib/CategoryTheory/EqToHom.lean |
3 |
1 |
['github-actions'] |
erdOne assignee:erdOne |
21-34931 21 days ago |
31-82920 1 month ago |
32-72802 32 days |
28375 |
euprunin author:euprunin |
chore(Analysis/SpecialFunctions/Pow): golf entire `rpow_lt_rpow_of_exponent_neg`, `rpow_le_rpow_of_exponent_nonpos`, `rpow_le_of_le_log` and `rpow_lt_of_lt_log` |
---
[](https://gitpod.io/from-referrer/)
|
t-analysis |
8/22 |
Mathlib/Analysis/SpecialFunctions/Pow/Real.lean |
1 |
2 |
['JonBannon', 'Ruben-VandeVelde', 'github-actions'] |
urkud assignee:urkud |
21-34927 21 days ago |
30-23414 30 days ago |
30-23456 30 days |
28378 |
euprunin author:euprunin |
chore(Algebra): golf entire `eq_lift_comp_mkRingHom` and `eq_liftAlgHom_comp_mkAlgHom` |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
4/8 |
Mathlib/Algebra/RingQuot.lean |
1 |
1 |
['github-actions'] |
mariainesdff assignee:mariainesdff |
21-34926 21 days ago |
30-22771 30 days ago |
30-22813 30 days |
28399 |
Ruben-VandeVelde author:Ruben-VandeVelde |
feat: ring-theoretic fractions in Rat |
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory |
47/0 |
Mathlib.lean,Mathlib/RingTheory/Localization/Rat.lean |
2 |
1 |
['github-actions'] |
robertylewis assignee:robertylewis |
21-34925 21 days ago |
30-7861 30 days ago |
30-7905 30 days |
28473 |
EtienneC30 author:EtienneC30 |
feat: toLp and ofLp are analytic |
---
[](https://gitpod.io/from-referrer/)
|
t-analysis |
42/0 |
Mathlib.lean,Mathlib/Analysis/Analytic/WithLp.lean |
2 |
1 |
['github-actions'] |
hrmacbeth assignee:hrmacbeth |
21-34922 21 days ago |
28-75496 28 days ago |
28-75477 28 days |
27990 |
kckennylau author:kckennylau |
feat(Counterexamples): a nontrivial valuation with discrete topology |
This file constructs a valuation on `K[X]` satisfying `IsValuativeTopology K[X] ∧ Nonempty (valuation K[X]).RankOne ∧ IsNontrivial K[X] ∧ DiscreteTopology K[X]`, and proves that `IsValuativeTopology F ∧ IsNontrivial F ∧ DiscreteTopology F` is not possible if `F` is a field.
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory |
172/0 |
Counterexamples.lean,Counterexamples/DiscreteTopologyWithNontrivialValuation.lean |
2 |
n/a |
['github-actions', 'grunweg', 'kckennylau', 'pechersky'] |
nobody |
21-20010 21 days ago |
unknown |
unknown |
24612 |
Paul-Lez author:Paul-Lez |
feat(Tactic/ImportDiff): add `#import_diff` command |
This PR adds the `#import_diff` command, which lists new transitive imports added by extending the list of imports of a file. The aim of this command is to help with debugging large import changes.
---
[](https://gitpod.io/from-referrer/)
|
will-close-soon
t-meta
awaiting-author
|
35/0 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/ImportDiff.lean |
3 |
9 |
['Paul-Lez', 'adomani', 'github-actions', 'joneugster'] |
adomani and joneugster assignee:joneugster assignee:adomani |
20-79958 20 days ago |
98-48486 3 months ago |
2-61262 2 days |
28807 |
alreadydone author:alreadydone |
experiment: Submodule with SMul only (no Semiring) |
---
`SubMulAction` already takes `SMul`.
TODO: relax typeclass requirements of `Ideal` as well.
[](https://gitpod.io/from-referrer/)
|
bench-after-CI
t-algebra
awaiting-CI
label:t-algebra$ |
54/42 |
Mathlib/Algebra/Module/Submodule/Defs.lean |
1 |
1 |
['github-actions'] |
nobody |
20-75936 20 days ago |
20-75947 20 days ago |
0-0 0 seconds |
28812 |
yury-harmonic author:yury-harmonic |
feat(PNat/Factors): add attrs and lemmas |
---
[](https://gitpod.io/from-referrer/)
|
t-data
new-contributor
|
42/0 |
Mathlib/Data/PNat/Factors.lean |
1 |
1 |
['github-actions'] |
nobody |
20-70524 20 days ago |
20-70680 20 days ago |
20-70718 20 days |
27245 |
rirarika author:rirarika |
feat: multivariate polynomial ring properties about irreducibility |
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-algebra
label:t-algebra$ |
88/0 |
Mathlib.lean,Mathlib/Algebra/MvPolynomial/Irreducible.lean |
2 |
5 |
['alreadydone', 'github-actions', 'mbkybky'] |
alreadydone assignee:alreadydone |
20-67713 20 days ago |
57-9759 1 month ago |
57-9799 57 days |
27479 |
iu-isgood author:iu-isgood |
feat: Abel's Binomial Theorem |
We have formalized Abel's Binomial Theorem as part of an REU project. There are a few remaining sorrys, but we will finish them soon. I will edit this PR message later according to community rules.
---
[](https://gitpod.io/from-referrer/)
|
t-data
new-contributor
awaiting-author
|
326/0 |
Mathlib/Data/Nat/Choose/AbelBinomial.lean |
1 |
28 |
['ElifUskuplu', 'FrankieNC', 'github-actions', 'iu-isgood'] |
nobody |
20-67695 20 days ago |
44-45592 1 month ago |
0-533 8 minutes |
25907 |
mans0954 author:mans0954 |
feat: low order roots of unity |
This PR continues the work from #25470.
Original PR: https://github.com/leanprover-community/mathlib4/pull/25470 |
t-algebra label:t-algebra$ |
182/0 |
Mathlib/Algebra/CharP/Invertible.lean,Mathlib/RingTheory/RootsOfUnity/Complex.lean |
2 |
2 |
['github-actions', 'mans0954'] |
kim-em assignee:kim-em |
20-67675 20 days ago |
89-80366 2 months ago |
89-80412 89 days |
25700 |
grunweg author:grunweg |
feat: lint upon uses of the `mono` tactic |
suggesting to use `gcongr` instead.
In general, `mono` is unmaintained, was only partially ported --- and gcongr at this point is more featureful, actively developed and has a nicer user interface. The topic was also discussed [on zulip](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Porting.20note.3A.20Fixing.20up.20.60mono.60/with/445125798).
---
TODO: update the linter wording, fix its implementation and wait until tests pass
- [ ] depends on: #25698
[](https://gitpod.io/from-referrer/)
|
t-linter
RFC
please-adopt
|
15/0 |
MathlibTest/DeprecatedSyntaxLinter.lean,MathlibTest/Monotonicity.lean |
2 |
3 |
['github-actions', 'grunweg', 'mathlib4-dependent-issues-bot'] |
nobody |
20-67340 20 days ago |
20-67382 20 days ago |
72-55831 72 days |
28215 |
5hv5hvnk author:5hv5hvnk |
Draft PR, for Strong and Weak connectivity for Digraphs |
strong and weak connectivity in Digraphs
---
Should resolve a part of issue #26771
Main additions in the PR:
1. Walks in Digraphs (Walk.lean)
- Basic walk structure with start and end vertices
- Support for walk operations: append, reverse, length
- Support functions: getVert, copy, support
2. Walk Decompositions (WalkDecomp.lean)
- takeUntil and dropUntil functions to split walks
- rotate operation for loop walks
- Theorems relating to walk decomposition properties
3. Subgraphs (subgraph.lean)
- Subgraph structure for digraphs
- Induced and spanning subgraph predicates
- Lattice structure (sup, inf, top, bot)
- Coercion to standalone digraphs
4. Paths (Paths.lean)
- Trail, Path, Circuit, Cycle definitions
- Path structure with no repeating vertices
- Theorems relating different path types
- Basic connectivity definitions (reachable, weakly/strongly connected)
5. Connectivity (Connected.lean)
- Reachability relations and properties
- Strong and weak connectivity definitions
- Connected component types:
- StronglyConnectedComponent
- WeaklyConnectedComponent
- ConnectedComponent
- Component properties and equivalence relations
-->
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-combinatorics
awaiting-author
|
1216/0 |
Mathlib/Combinatorics/Digraph/Connected.lean,Mathlib/Combinatorics/Digraph/Paths.lean,Mathlib/Combinatorics/Digraph/Subgraph.lean,Mathlib/Combinatorics/Digraph/Walk.lean,Mathlib/Combinatorics/Digraph/WalkDecomp.lean |
5 |
3 |
['github-actions', 'grunweg'] |
nobody |
20-66278 20 days ago |
20-66278 20 days ago |
12-41939 12 days |
28821 |
yury-harmonic author:yury-harmonic |
feat(SimpleGraph/Finite): add lemmas |
`simpNF` complains because `*Finset` are `abbrev`s.
---
[](https://gitpod.io/from-referrer/)
|
t-combinatorics |
24/1 |
Mathlib/Combinatorics/SimpleGraph/Finite.lean |
1 |
1 |
['github-actions'] |
nobody |
20-50707 20 days ago |
20-50757 20 days ago |
0-0 0 seconds |
28195 |
gasparattila author:gasparattila |
feat: separating a convex compact set and its neighborhood with a polytope |
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-analysis
|
26/1 |
Mathlib/Analysis/Normed/Affine/Convex.lean |
1 |
2 |
['FrankieNC', 'github-actions'] |
sgouezel assignee:sgouezel |
20-34899 20 days ago |
33-50833 1 month ago |
33-50884 33 days |
28439 |
euprunin author:euprunin |
chore(LinearAlgebra/Matrix/Determinant): golf entire `det_eq_zero_of_not_linearIndependent_rows` |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
1/5 |
Mathlib/LinearAlgebra/Matrix/Determinant/Basic.lean |
1 |
1 |
['github-actions'] |
mariainesdff assignee:mariainesdff |
20-34895 20 days ago |
29-51942 29 days ago |
29-51986 29 days |
28531 |
Ruben-VandeVelde author:Ruben-VandeVelde |
chore: remove Cardinal imports from Topology.Algebra.InfiniteSum.Group |
---
[](https://gitpod.io/from-referrer/)
|
|
51/15 |
Mathlib.lean,Mathlib/Analysis/BoxIntegral/UnitPartition.lean,Mathlib/Analysis/Normed/Group/Pointwise.lean,Mathlib/Analysis/Normed/Module/Convex.lean,Mathlib/Analysis/SpecificLimits/Basic.lean,Mathlib/Topology/Algebra/InfiniteSum/Const.lean,Mathlib/Topology/Algebra/InfiniteSum/Group.lean,Mathlib/Topology/Algebra/InfiniteSum/NatInt.lean,Mathlib/Topology/Algebra/InfiniteSum/Order.lean,Mathlib/Topology/Algebra/InfiniteSum/Real.lean,Mathlib/Topology/Category/Stonean/Basic.lean,Mathlib/Topology/Instances/ENNReal/Lemmas.lean,Mathlib/Topology/Instances/NNReal/Lemmas.lean,Mathlib/Topology/MetricSpace/HausdorffDistance.lean,Mathlib/Topology/MetricSpace/Thickening.lean,Mathlib/Topology/PartitionOfUnity.lean |
16 |
4 |
['Ruben-VandeVelde', 'YaelDillies', 'github-actions'] |
TwoFX assignee:TwoFX |
20-34891 20 days ago |
27-45743 27 days ago |
27-45723 27 days |
28766 |
yury-harmonic author:yury-harmonic |
feat(Nat/Factorial): add tail-recursive versions |
---
[](https://gitpod.io/from-referrer/)
|
t-data
new-contributor
|
58/1 |
Mathlib/Data/Nat/Factorial/Basic.lean |
1 |
1 |
['github-actions', 'plp127'] |
nobody |
20-34203 20 days ago |
22-14291 22 days ago |
22-14338 22 days |
28837 |
yury-harmonic author:yury-harmonic |
feat(ValMinAbs): add lemmas |
---
[](https://gitpod.io/from-referrer/)
|
t-data |
24/6 |
Mathlib/Data/ZMod/ValMinAbs.lean |
1 |
1 |
['github-actions'] |
nobody |
20-12079 20 days ago |
20-12089 20 days ago |
20-12125 20 days |
27965 |
grunweg author:grunweg |
feat: verify that file names contain no forbidden characters |
Follow-up to #27588: Windows also forbids certain characters in file names.
I snuck in a change to also disallow `!` (which causes problems on Nix OS) and
`.` (i.e., #27944) --- that would have caught the error in #27796, and may indicate confusion of file and module names.
---
[](https://gitpod.io/from-referrer/)
|
file-removed
t-linter
maintainer-merge
|
72/42 |
Mathlib/Tactic/Linter/TextBased.lean,MathlibTest/ForbiddenModuleNames.lean,MathlibTest/ForbiddenWindows.lean,scripts/lint-style.lean |
4 |
12 |
['YaelDillies', 'adomani', 'euprunin', 'github-actions', 'grunweg'] |
joneugster assignee:joneugster |
19-62529 19 days ago |
38-60216 1 month ago |
39-6095 39 days |
28604 |
alreadydone author:alreadydone |
chore(Algebra/Ring/Defs): add two classes (minimally invasive version) |
Add the missing `NonAssocComm(Semi)ring` classes and add some missing instances between existing classes. Contrary to #28532, the approach here doesn't add any new `extends`.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
WIP
label:t-algebra$ |
59/17 |
Mathlib/Algebra/Colimit/DirectLimit.lean,Mathlib/Algebra/Ring/Defs.lean,Mathlib/LinearAlgebra/CliffordAlgebra/Basic.lean |
3 |
15 |
['alreadydone', 'github-actions', 'leanprover-bot'] |
nobody |
19-56020 19 days ago |
24-84732 24 days ago |
0-59042 16 hours |
28868 |
yury-harmonic author:yury-harmonic |
feat(Positive): add `OfNat` instance |
Also fix defeq for `Div` in the `Group` instance.
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebra
label:t-algebra$ |
41/13 |
Mathlib/Algebra/Order/Positive/Field.lean,Mathlib/Algebra/Order/Positive/Ring.lean,Mathlib/Data/PNat/Defs.lean |
3 |
2 |
['github-actions', 'yury-harmonic'] |
nobody |
19-54105 19 days ago |
19-56928 19 days ago |
19-56972 19 days |
27357 |
jcreedcmu author:jcreedcmu |
feat(Algebra/Module/Submodule): add `submoduleMap` for isometries |
Per [discussion on Zulip](https://leanprover.zulipchat.com/#narrow/channel/217875-Is-there-code-for-X.3F/topic/Analog.20of.20LinearEquiv.2EsubmoduleMap.20for.20AffineIsometryEquiv.3F), add a version of `.submoduleMap` for `LinearIsometry` and `LinearIsometryEquiv` by analogy with `LinearMap.submoduleMap` and `LinearEquiv.submoduleMap`.
--- |
new-contributor
t-algebra
label:t-algebra$ |
36/0 |
Mathlib/Analysis/Normed/Operator/LinearIsometry.lean |
1 |
24 |
['Ruben-VandeVelde', 'dagurtomas', 'eric-wieser', 'github-actions', 'jcreedcmu', 'themathqueen'] |
dagurtomas assignee:dagurtomas |
19-47637 19 days ago |
19-47637 19 days ago |
49-29945 49 days |
28884 |
kim-em author:kim-em |
chore: deprecate ShiftLeft Int instance |
This PR proposes deprecating the `ShiftLeft Int` instance (which allows bit-shifting an integer by an integer), and similarly for `ShiftRight`.
These are unused in Mathlib.
I'm happy if someone wants to keep this, but I would ask that they:
* fix the doc-strings to explain what happens for negative shifts
* ~~restores the theorem `Int.shiftLeft_add` which I've commented out on `nightly-testing` (and then revert b33c9d7aaea on `nightly-testing`).~~
* ideally but optionally, complete the API, e.g. reducing shifts by casts back to shifts by a Nat |
t-data |
22/2 |
Mathlib/Data/Int/Bitwise.lean |
1 |
4 |
['eric-wieser', 'github-actions', 'kim-em'] |
nobody |
19-38217 19 days ago |
19-42768 19 days ago |
19-42805 19 days |
27944 |
grunweg author:grunweg |
feat: lint module names with a period |
This would have caught the mis-placed file in #27796.
---
[](https://gitpod.io/from-referrer/)
|
t-linter |
16/0 |
Mathlib/Tactic/Linter/TextBased.lean,scripts/lint-style.lean |
2 |
2 |
['github-actions', 'grunweg'] |
joneugster assignee:joneugster |
19-34897 19 days ago |
39-60366 1 month ago |
39-60347 39 days |
28132 |
dupuisf author:dupuisf |
feat: preliminary `grind` tags for `IsUnit` |
This PR adds preliminary `grind` tags for the `IsUnit` predicate.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
61/17 |
Mathlib/Algebra/Group/Action/Units.lean,Mathlib/Algebra/Group/Units/Defs.lean,Mathlib/Algebra/GroupWithZero/Units/Basic.lean,Mathlib/Algebra/Ring/Units.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Order.lean,Mathlib/Analysis/SpecialFunctions/ContinuousFunctionalCalculus/Rpow/Basic.lean |
6 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
kim-em assignee:kim-em |
19-34896 19 days ago |
28-31244 28 days ago |
28-31225 28 days |
28325 |
pechersky author:pechersky |
feat(WithZeroTopology): `locallyCompactSpace_iff_locallyFiniteOrder_units` |
On the way to golf/generalize the proof that
locally compact valued fields have locally finite valuation groups as embodied in
`Valued.integer.locallyFiniteOrder_units_mrange_of_isCompact_integer` ]
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-order
t-topology
|
160/2 |
Mathlib/Topology/Algebra/GroupWithZero.lean,Mathlib/Topology/Algebra/WithZeroTopology.lean,Mathlib/Topology/Compactness/Compact.lean |
3 |
1 |
['github-actions'] |
PatrickMassot assignee:PatrickMassot |
19-34893 19 days ago |
31-17109 1 month ago |
31-19816 31 days |
27207 |
pechersky author:pechersky |
feat(Topology/WithVal): ValuativeRel (WithVal v) |
with a helper valuation defined that does not pierce defeq
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-topology
label:t-algebra$ |
20/1 |
Mathlib/Topology/Algebra/Valued/WithVal.lean |
1 |
7 |
['alreadydone', 'github-actions', 'mathlib4-merge-conflict-bot', 'pechersky', 'smmercuri'] |
alreadydone assignee:alreadydone |
19-27833 19 days ago |
19-27949 19 days ago |
52-80628 52 days |
26988 |
YaelDillies author:YaelDillies |
feat(Rel): more API |
Some of this API already exists in `Topology.UniformSpace.Defs` but not spelled with `SetRel`, some of it was written for #24173.
---
`Topology.UniformSpace.Defs` will be refactored to use these new lemmas in #23181.
[](https://gitpod.io/from-referrer/)
|
t-data |
182/8 |
Mathlib/Combinatorics/SimpleGraph/Basic.lean,Mathlib/Data/Rel.lean |
2 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
19-17844 19 days ago |
31-15941 1 month ago |
63-76578 63 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
awaiting-author
|
187/0 |
Mathlib.lean,Mathlib/Combinatorics/SimpleGraph/Cycle.lean |
2 |
41 |
['IvanRenison', 'github-actions', 'vlad902'] |
kmill assignee:kmill |
19-9354 19 days ago |
19-9354 19 days ago |
123-22718 123 days |
28329 |
pechersky author:pechersky |
feat(RingTheory/Valuation): generalize CommGroupWithZero on mrange to MonoidWithZeroHom |
Before, they were only for Valuation, but that is too restricted
---
[](https://gitpod.io/from-referrer/)
|
maintainer-merge
t-order
t-algebra
label:t-algebra$ |
77/27 |
Mathlib.lean,Mathlib/Algebra/GroupWithZero/Range.lean,Mathlib/Algebra/GroupWithZero/Submonoid/Instances.lean,Mathlib/RingTheory/Valuation/Archimedean.lean,Mathlib/RingTheory/Valuation/Basic.lean |
5 |
10 |
['YaelDillies', 'eric-wieser', 'github-actions', 'pechersky'] |
YaelDillies assignee:YaelDillies |
19-1758 19 days ago |
19-19465 19 days ago |
27-47819 27 days |
27963 |
ShreckYe author:ShreckYe |
feat(Algebra/GCDMonoid): add some theorems related to divisibility and `lcm` for both `GCDMonoid` and `Nat` |
While working on formalizing some math olympiad problems, I found that the theorem `dvd_lcm : p ∣ lcm a b ↔ p ∣ a ∨ p ∣ b` is missing in Mathlib. So I added this along with some other related theorems. These theorems are simlilar to those related to divisibility and multiplication (`dvd_mul` as compared to `dvd_lcm` for example), as commented in the doc strings. |
new-contributor
t-algebra
label:t-algebra$ |
102/0 |
Mathlib.lean,Mathlib/Algebra/GCDMonoid/Basic.lean,Mathlib/Data/Nat/GCD/Basic.lean,Mathlib/Data/Nat/GCD/Prime.lean |
4 |
29 |
['Ruben-VandeVelde', 'ShreckYe', 'github-actions', 'themathqueen'] |
erdOne assignee:erdOne |
18-71591 18 days ago |
24-74806 24 days ago |
32-78448 32 days |
28376 |
euprunin author:euprunin |
chore(Analysis/Calculus/Deriv): golf entire `differentiableAt_comp_const_add` |
---
[](https://gitpod.io/from-referrer/)
|
t-analysis
awaiting-author
|
2/6 |
Mathlib/Analysis/Calculus/Deriv/Add.lean |
1 |
1 |
['github-actions', 'loefflerd'] |
nobody |
18-52891 18 days ago |
18-52891 18 days ago |
11-56866 11 days |
23835 |
chrisflav author:chrisflav |
feat(Topology): cardinality of connected components is bounded by cardinality of fiber |
We show that if `f : X → Y` is an open and closed map to `Y` and `Y` is connected, the number of connected
components of `X` is bounded by the cardinality of the fiber of any point. In particular, if `Y` has finitely many connected components and `f` finite fibers, also `X` as finitely many connected components.
From Pi1.
---
- [x] depends on: #23849
[](https://gitpod.io/from-referrer/)
|
t-topology |
242/1 |
Mathlib.lean,Mathlib/Data/Set/Lattice.lean,Mathlib/SetTheory/Cardinal/Finite.lean,Mathlib/Topology/Clopen.lean,Mathlib/Topology/Connected/CardComponents.lean,Mathlib/Topology/Connected/Clopen.lean |
6 |
5 |
['chrisflav', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
grunweg assignee:grunweg |
18-34925 18 days ago |
25-78474 25 days ago |
27-72505 27 days |
27824 |
ChrisHughes24 author:ChrisHughes24 |
feat(Calculus): exists_gt_of_deriv_pos and variants |
---
I created a new file for this as I anticipate there will be many lemmas relating derivatives and monotonicity in future. Some lemmas relating deriviatives to monotonicity are already in mathlib and should maybe moved to the file (e.g. docs#HasDerivWithinAt.nonneg_of_monotoneOn).
I stated them in as much generality as I could, copying the generality of `HasDerivWithinAt.nonneg_of_monotoneOn`.
- [x] depends on: #28039
[](https://gitpod.io/from-referrer/)
|
t-analysis |
85/0 |
Mathlib.lean,Mathlib/Analysis/Calculus/Deriv/Order.lean |
2 |
29 |
['ChrisHughes24', 'EtienneC30', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
hrmacbeth assignee:hrmacbeth |
18-34922 18 days ago |
28-65122 28 days ago |
32-82817 32 days |
28487 |
euprunin author:euprunin |
chore(RingTheory): golf entire `smul_eq_zero_of_mem`, `hasEval`, `eq_of_prod_eq_prod` and `isIntegral_of_mem_ringOfIntegers` |
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory |
7/16 |
Mathlib/RingTheory/Extension/Basic.lean,Mathlib/RingTheory/PowerSeries/Substitution.lean,Mathlib/RingTheory/UniqueFactorizationDomain/FactorSet.lean,Mathlib/RingTheory/Valuation/AlgebraInstances.lean |
4 |
1 |
['github-actions'] |
erdOne assignee:erdOne |
18-34916 18 days ago |
28-65901 28 days ago |
28-65944 28 days |
28489 |
joelriou author:joelriou |
feat(CategoryTheory): weaken assumptions for the stability of the left lifting property under transfinite compositions |
This PR introduces two predicates `HasLiftingPropertyFixedBot/Top` which assert the existence of a lifting in squares when the left/right/top (resp. left/right/bottom) morphisms are fixed. (This weakens the `HasLiftingProperty` class which assumes there is a lifting when we only fix the left and right morphisms.)
The `HasLiftingPropertyFixedTop` variant shall be used in the study of the homotopy theory of Kan complexes. Hopefully, the `HasLiftingPropertyFixedBot` variant will be used in the formalization of the model category structure on simplicial sets: this is the reason why this PR also weakens the assumptions in the proof that the left lifting property with respect to certain morphisms is stable under transfinite composition.
---
[](https://gitpod.io/from-referrer/)
|
t-category-theory |
28/2 |
Mathlib/CategoryTheory/LiftingProperties/Basic.lean,Mathlib/CategoryTheory/SmallObject/TransfiniteCompositionLifting.lean |
2 |
1 |
['github-actions'] |
b-mehta assignee:b-mehta |
18-34916 18 days ago |
28-63045 28 days ago |
28-63026 28 days |
27155 |
Pjotr5 author:Pjotr5 |
feat: Shearer's bound on the independence number of triangle free graphs |
I added the file IndependenceNumber.lean to the Mathlib.Combinatorics.SimpleGraph.Triangle folder. It contains a proof of a theorem by Shearer on the independence number of triangle-free graphs . I was told this might be useful to add to Mathlib a Zullip thread linked [here](https://leanprover.zulipchat.com/#narrow/channel/217875-Is-there-code-for-X.3F/topic/Convexity.20of.20a.20specific.20function/with/510469526).
I tried to comply as much as I could with the Mathlib style guide, but I realise that there is probably still a significant amount of editing to be done. For one thing: there are probably some lemmas and theorems in there that might be better suited in other files, but since this is my first PR I though I would all put it in one file before starting to edit a bunch of files.
I was also advised to split up the file into multiple smaller PRs, but since everything is basically serving this one proof I could not really find a natural way to do that.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-combinatorics
awaiting-author
|
1266/0 |
Mathlib.lean,Mathlib/Combinatorics/SimpleGraph/Triangle/IndependenceNumber.lean |
2 |
9 |
['Pjotr5', 'github-actions', 'grunweg'] |
nobody |
18-12322 18 days ago |
20-66931 20 days ago |
39-17587 39 days |
28445 |
mitchell-horner author:mitchell-horner |
feat: `one_sub_one_div_cast_*` theorems |
---
Needed for a proof of the Erdős-Stone-Simonovits theorem in future PR.
[](https://gitpod.io/from-referrer/)
|
t-data
t-algebra
t-number-theory
label:t-algebra$ |
18/0 |
Mathlib/Data/Nat/Cast/Order/Field.lean |
1 |
1 |
['github-actions'] |
nobody |
18-7583 18 days ago |
18-7583 18 days ago |
29-46100 29 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
awaiting-author
label:t-algebra$ |
10/0 |
Mathlib/LinearAlgebra/Matrix/NonsingularInverse.lean |
1 |
16 |
['eric-wieser', 'github-actions', 'madvorak', 'ocfnash'] |
nobody |
18-6232 18 days ago |
39-74609 1 month ago |
86-39206 86 days |
28149 |
Equilibris author:Equilibris |
feat: dcongr_heq |
`dcongr_heq` is very useful for proofs about typevecs as these are highly dependent
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-logic
|
14/0 |
Mathlib/Logic/Basic.lean |
1 |
13 |
['Equilibris', 'alexkeizer', 'fpvandoorn', 'github-actions', 'madvorak'] |
fpvandoorn assignee:fpvandoorn |
18-3926 18 days ago |
35-5318 1 month ago |
35-5360 35 days |
28350 |
themathqueen author:themathqueen |
feat(Algebra/Module/LinearMap): `range (f.smulRight x) = span {x}` |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
55/8 |
Mathlib.lean,Mathlib/Algebra/Module/LinearMap/Lemmas.lean,Mathlib/LinearAlgebra/Dual/Lemmas.lean,Mathlib/Topology/Algebra/Module/LinearMap.lean |
4 |
3 |
['Ruben-VandeVelde', 'github-actions', 'themathqueen'] |
dagurtomas assignee:dagurtomas |
18-3320 18 days ago |
18-3320 18 days ago |
30-69573 30 days |
27242 |
hugh-fox author:hugh-fox |
feat: add Gauss-like formula for sums of digit sums |
Adds `sum_digit_sum_base_pow_eq` to show a Gauss-like formula across sums of digit sums.
This relies on an additional two simp lemmas, named `digits_sum_eq_self`, `digits_sum_base_mul_cancel`.
Lastly, includes a specialization (which is a good bit simpler than the general formula) to base 10 named `sum_digit_sum_ten_pow_eq`.
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-data
new-contributor
awaiting-author
|
113/0 |
Mathlib/Data/Nat/Digits/Lemmas.lean |
1 |
5 |
['github-actions', 'hugh-fox', 'kckennylau'] |
nobody |
17-73691 17 days ago |
17-73691 17 days ago |
39-41606 39 days |
27047 |
YaelDillies author:YaelDillies |
feat: `MonoidHom.toAdditive''` as a `MulEquiv` |
From Toric
---
I haven't yet been very thorough with the new lemmas. I first want to hear thoughts about the names
[](https://gitpod.io/from-referrer/)
|
toric
t-algebra
label:t-algebra$ |
31/7 |
Mathlib/Algebra/Group/TypeTags/Hom.lean |
1 |
1 |
['github-actions'] |
adomani assignee:adomani |
17-70309 17 days ago |
62-15133 2 months ago |
62-46987 62 days |
26961 |
mariainesdff author:mariainesdff |
feat(RingTheory/PowerSeries/Substitution): add API |
Co-authored-by: @AntoineChambert-Loir
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
awaiting-author
|
62/1 |
Mathlib/RingTheory/PowerSeries/Basic.lean,Mathlib/RingTheory/PowerSeries/Substitution.lean |
2 |
12 |
['Ruben-VandeVelde', 'github-actions', 'mariainesdff', 'mattrobball'] |
mattrobball assignee:mattrobball |
17-66479 17 days ago |
17-66479 17 days ago |
47-20047 47 days |
28925 |
grunweg author:grunweg |
chore: remove `linear_combination'` tactic |
When `linear_combination` was refactored in #15899, the old code was kept as the `linear_combination'` tactic, for easier migration. The consensus of the zulip discussion ([#mathlib4 > Narrowing the scope of `linear_combination` @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Narrowing.20the.20scope.20of.20.60linear_combination.60/near/470237816)) was to wait, and "revisit this once people have experienced the various tactics in practice".
One year later, the old tactic has almost no uses: it is unused in mathlib; [searching on github](https://github.com/search?q=linear_combination%27%20path%3A*.lean&type=code) yields 37 hits --- all of which are in various forks of mathlib. Thus, removing this tactic seems appropriate.
---
Do not merge before the zulip discussion has concluded!
[](https://gitpod.io/from-referrer/)
|
file-removed
awaiting-zulip
|
0/564 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/LinearCombination'.lean,Mathlib/Tactic/Linter/UnusedTactic.lean,MathlibTest/linear_combination'.lean |
5 |
3 |
['euprunin', 'github-actions', 'grunweg'] |
nobody |
17-64073 17 days ago |
18-47806 18 days ago |
0-1 1 second |
25292 |
YaelDillies author:YaelDillies |
feat: the `ConvexCone` generated by a set |
Define `ConvexCone.copy` and `ConvexCone.hull` and use them to golf the `CompleteLattice` instance.
From Toric
---
- [x] depends on: #25291
[](https://gitpod.io/from-referrer/)
|
t-convex-geometry
toric
|
94/35 |
Mathlib/Analysis/Convex/Cone/Basic.lean,Mathlib/Geometry/Convex/Cone/Basic.lean |
2 |
8 |
['YaelDillies', 'b-mehta', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
17-48011 17 days ago |
48-454 1 month ago |
85-38777 85 days |
28768 |
yury-harmonic author:yury-harmonic |
feat(Data/Nat): define `Nat.nthRoot` |
Define `Nat.nthRoot n a` to be the `n`th root of a natural number `a`.
---
This is a dependency of a `norm_num` plugin that can handle `(8 : Real) ^ (2 / 3 : Real)`.
[](https://gitpod.io/from-referrer/)
|
t-data
new-contributor
|
218/0 |
Mathlib.lean,Mathlib/Data/Nat/NthRoot/Defs.lean,Mathlib/Data/Nat/NthRoot/Lemmas.lean |
3 |
16 |
['b-mehta', 'eric-wieser', 'github-actions', 'j-loreaux', 'yury-harmonic'] |
nobody |
17-47148 17 days ago |
21-20457 21 days ago |
21-61540 21 days |
27992 |
staroperator author:staroperator |
feat(Algebra): cancellation inheritance |
This PR:
1. adds `Is{Left,Right}Cancel{Add,Mul,MulZero}` instances for `{Add,Mul,MulZero}MemClass` etc.
2. duplicates such instances for `Subsemiring` and `Subalgebra`, following #27955 (which is for `Submonoid` and `Submodule`).
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
74/1 |
Mathlib.lean,Mathlib/Algebra/Algebra/Subalgebra/Basic.lean,Mathlib/Algebra/Group/Submonoid/Defs.lean,Mathlib/Algebra/Group/Subsemigroup/Defs.lean,Mathlib/Algebra/GroupWithZero/Submonoid/CancelMulZero.lean,Mathlib/Algebra/Module/Submodule/Defs.lean,Mathlib/Algebra/Ring/Subsemiring/Defs.lean |
7 |
7 |
['Vierkantor', 'eric-wieser', 'github-actions', 'mathlib4-merge-conflict-bot', 'staroperator'] |
alreadydone assignee:alreadydone |
17-34922 17 days ago |
32-43584 1 month ago |
38-53748 38 days |
26088 |
grunweg author:grunweg |
chore(Linter/DirectoryDependency): move forbidden directories into a JSON file |
This PR continues the work from #25406.
Original PR: https://github.com/leanprover-community/mathlib4/pull/25406 |
t-linter |
387/19 |
Mathlib/Tactic/Linter/DirectoryDependency.lean,scripts/README.md,scripts/forbiddenDirs.json |
3 |
3 |
['github-actions', 'grunweg', 'mathlib4-merge-conflict-bot'] |
nobody |
17-4881 17 days ago |
17-4901 17 days ago |
86-42243 86 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 |
6 |
['IvanRenison', 'github-actions', 'vlad902'] |
kmill assignee:kmill |
16-83560 16 days ago |
109-40686 3 months ago |
109-40736 109 days |
27261 |
Sebi-Kumar author:Sebi-Kumar |
feat(Topology): add definition for subpaths |
Define subpaths as restrictions of paths to subintervals, reparameterized to have domain
`[0, 1]` and possibly with a reverse of direction. Prove their basic properties.
This serves as an alternative to `Path.truncate` which is useful for the explicit construction of certain homotopies, in particular regarding the concatenation of subpaths.
---
To provide additional context, this is my first time contributing to Mathlib,
and I am doing so as a part of the Fields Undergraduate Summer Research Program
hosted at Western University.
My intention for this file is for it to be used when proving that the fundamental group of the sphere is trivial (following the proof from Hatcher's "Algebraic Topology").
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-topology
awaiting-author
|
146/0 |
Mathlib.lean,Mathlib/Topology/Subpath.lean |
2 |
24 |
['ADedecker', 'FrankieNC', 'Sebi-Kumar', 'github-actions', 'themathqueen', 'wwylele'] |
ADedecker assignee:ADedecker |
16-75131 16 days ago |
22-43622 22 days ago |
34-15767 34 days |
26644 |
kckennylau author:kckennylau |
feat(SetTheory/ZFC): Define the language of sets and state the ZFC axioms |
---
[](https://gitpod.io/from-referrer/)
|
t-set-theory
awaiting-author
|
381/0 |
Mathlib.lean,Mathlib/SetTheory/ZFC/Axioms.lean,docs/references.bib |
3 |
49 |
['b-mehta', 'digama0', 'github-actions', 'kckennylau', 'leanprover-community-bot-assistant', 'staroperator', 'vihdzp'] |
b-mehta assignee:b-mehta |
16-69446 16 days ago |
19-61525 19 days ago |
40-53883 40 days |
26914 |
quangvdao author:quangvdao |
feat(Data/PFunctor/Univariate): more definitions for univariate `PFunctor` |
This PR defines several basic definitions of `PFunctor`, including zero, one, constants, monomials, coproduct (sum), product, sigma, pi, tensor product, universe lifting, and equivalence.
We also add: (1) simple lemmas connecting the basic definitions, (2) an automatically derived ext lemma for `PFunctor` via `@[ext]` attribute
Some things I'm not clear on:
- I define `HAdd` and `HMul` instances for coproduct and product of poly functors having different universe levels. Should I also define `Add` and `Mul` instances for poly functors having the same universe level?
- Is it ok to define notation for tensor product, i.e. `@[inherit_doc] scoped infixr:80 " ⊗ " => tensor`? I'm worried it might clash with other notation.
- Need a double-check on the priority of notation.
Some future definitions to add:
- Various equivalences arising from arithmetic identities, e.g., `P + 0 ≃ₚ P`.
- Definitions of Lenses and Charts (each of them will be a file or even a folder)
- Exponential objects (corresponding to both `prod` and `tensor`)
---
[](https://gitpod.io/from-referrer/)
|
t-data |
144/5 |
Mathlib/Data/PFunctor/Univariate/Basic.lean |
1 |
19 |
['alexkeizer', 'eric-wieser', 'github-actions', 'quangvdao'] |
eric-wieser assignee:eric-wieser |
16-68276 16 days ago |
66-35983 2 months ago |
66-36025 66 days |
29030 |
b-mehta author:b-mehta |
feat(Combinatorics): prove the Rado selection lemma |
Prove the Rado selection lemma, a generic result useful to prove a variety of compactness results in combinatorics. This generalises Konig's infinity lemma, and the de Bruijn-Erdos theorem, and allows the former to be conveniently stated in the language of sets rather than categories.
This is a draft PR for now, since the imports are not correct and the names need fixing.
---
[](https://gitpod.io/from-referrer/)
|
t-combinatorics |
80/0 |
Mathlib/Combinatorics/SimpleGraph/DeBruijnErdos.lean |
1 |
1 |
['github-actions'] |
nobody |
16-63507 16 days ago |
16-63678 16 days ago |
0-0 0 seconds |
26648 |
eric-wieser author:eric-wieser |
chore(TensorProduct): remove more `suppress_compilation`s |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
blocked-by-core-PR
label:t-algebra$ |
3/7 |
Mathlib/LinearAlgebra/CliffordAlgebra/Prod.lean,Mathlib/LinearAlgebra/TensorProduct/Graded/External.lean,Mathlib/LinearAlgebra/TensorProduct/Graded/Internal.lean |
3 |
4 |
['eric-wieser', 'github-actions', 'leanprover-bot'] |
nobody |
16-63369 16 days ago |
16-63369 16 days ago |
3-19989 3 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 |
25 |
['YaelDillies', 'b-mehta', 'eric-wieser', 'github-actions', 'grunweg', 'kkytola', 'mathlib4-dependent-issues-bot', 'urkud'] |
alreadydone assignee:alreadydone |
16-62552 16 days ago |
124-59917 4 months ago |
172-25732 172 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
awaiting-author
|
319/0 |
Mathlib.lean,Mathlib/Algebra/BigOperators/Group/Finset/Disjoint.lean,Mathlib/Algebra/Module/ZLattice/Summable.lean,Mathlib/Order/Disjointed.lean |
4 |
3 |
['github-actions', 'wwylele'] |
fpvandoorn assignee:fpvandoorn |
16-62360 16 days ago |
16-62360 16 days ago |
76-21393 76 days |
28056 |
grunweg author:grunweg |
wip: existence of Riemannian metrics |
Work in progress: will require the material of #26221 (orthonormal frames), hence first be developed there.
---
- [x] depends on: #26875
- [x] depends on: #28046 (just nice to have, not strictly necessary)
[](https://gitpod.io/from-referrer/)
|
t-differential-geometry
WIP
|
785/0 |
Mathlib.lean,Mathlib/Geometry/Manifold/ExistsRiemannianMetric.lean,Mathlib/Geometry/Manifold/ExistsRiemannianMetric2.lean,Mathlib/Geometry/Manifold/VectorBundle/Riemannian.lean |
4 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
16-58160 16 days ago |
16-58233 16 days ago |
0-0 0 seconds |
26885 |
pechersky author:pechersky |
feat(Topology/ValuativeRel): ValuativeTopology 𝒪[K] |
and even when not a field, `ValuativeRel 𝒪[K]`
This is an example of something achievable with the new declarations that wasn't possible with Valued
Such that we can discuss the valuations on the subring without always using coercions
But to achieve this, one needs some juggling of the value groups
---
[](https://gitpod.io/from-referrer/)
- [x] depends on: #26834
|
t-algebra
t-topology
t-number-theory
label:t-algebra$ |
73/0 |
Mathlib/RingTheory/Valuation/ValuativeRel/Basic.lean,Mathlib/Topology/Algebra/Valued/ValuativeRel.lean |
2 |
6 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
alreadydone assignee:alreadydone |
16-55237 16 days ago |
16-55257 16 days ago |
66-40269 66 days |
27163 |
pechersky author:pechersky |
feat(Topology/ValuativeRel): of and to basis of compatible valuations |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-topology
t-number-theory
label:t-algebra$ |
205/25 |
Mathlib/RingTheory/Valuation/ValuativeRel/Basic.lean,Mathlib/Topology/Algebra/Valued/ValuativeRel.lean |
2 |
27 |
['github-actions', 'kckennylau', 'mathlib4-merge-conflict-bot', 'pechersky'] |
alreadydone assignee:alreadydone |
16-55105 16 days ago |
16-55126 16 days ago |
59-32213 59 days |
28490 |
euprunin author:euprunin |
chore: golf entire `epi_of_cokernel_π_eq_zero`, `bottom_row_coprime`, `congr_of_eventuallyEq` and `Invertible.congr` |
---
[](https://gitpod.io/from-referrer/)
|
|
8/12 |
Mathlib/Algebra/Group/Invertible/Defs.lean,Mathlib/CategoryTheory/Abelian/Basic.lean,Mathlib/NumberTheory/Modular.lean,Mathlib/Topology/ContinuousOn.lean |
4 |
1 |
['github-actions'] |
kex-y assignee:kex-y |
16-34918 16 days ago |
28-61364 28 days ago |
28-61344 28 days |
22662 |
plp127 author:plp127 |
feat: Localization.Away.lift (computably) |
This PR adds `Localization.Away.lift'` and `Localization.Away.lift`, computable alternatives to `Localization.awayLift`.
---
- [x] depends on: #24791
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
74/0 |
Mathlib/RingTheory/Localization/Away/Basic.lean |
1 |
17 |
['eric-wieser', 'github-actions', 'grunweg', 'mathlib4-dependent-issues-bot', 'plp127', 'vihdzp'] |
mariainesdff assignee:mariainesdff |
16-34682 16 days ago |
124-39297 4 months ago |
190-39276 190 days |
24373 |
YaelDillies author:YaelDillies |
refactor: golf `modularCharacter` |
... using the lessons learned from `distribHaarChar`. Unfortunately, the two setups can't quite be unified because we are lacking an additive version of `MulDistribMulAction`.
---
[](https://gitpod.io/from-referrer/)
|
t-measure-probability
awaiting-CI
|
77/45 |
Mathlib/MeasureTheory/Group/MeasurableEquiv.lean,Mathlib/MeasureTheory/Group/Measure.lean,Mathlib/MeasureTheory/Group/ModularCharacter.lean,Mathlib/MeasureTheory/Integral/Bochner/Basic.lean,Mathlib/MeasureTheory/Measure/Haar/Unique.lean |
5 |
4 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-merge-conflict-bot'] |
nobody |
16-17464 16 days ago |
16-17490 16 days ago |
0-0 0 seconds |
24383 |
YaelDillies author:YaelDillies |
feat: distributive Haar characters of `ℝ` and `ℂ` |
Compute `distribHaarChar` in the case of the actions of `ℝˣ` on `ℝ` and of `ℂˣ` on `ℂ`.
The file I'm moving was added two days ago and is not yet used in FLT.
From FLT
---
[](https://gitpod.io/from-referrer/)
|
file-removed
FLT
t-measure-probability
awaiting-CI
WIP
|
205/78 |
Mathlib.lean,Mathlib/Algebra/BigOperators/GroupWithZero/Action.lean,Mathlib/Algebra/Group/Action/BigOperators.lean,Mathlib/MeasureTheory/Measure/Haar/DistribChar/Basic.lean,Mathlib/MeasureTheory/Measure/Haar/DistribChar/Complex.lean,Mathlib/MeasureTheory/Measure/Haar/DistribChar/Real.lean,Mathlib/MeasureTheory/Measure/Lebesgue/Basic.lean,Mathlib/MeasureTheory/Measure/Lebesgue/EqHaar.lean |
8 |
21 |
['YaelDillies', 'github-actions', 'kbuzzard', 'leanprover-community-bot-assistant', 'mathlib4-merge-conflict-bot', 'sgouezel'] |
nobody |
16-17278 16 days ago |
16-17301 16 days ago |
8-77637 8 days |
29010 |
grunweg author:grunweg |
chore: more tests for field_simp features and edge cases |
---
[](https://gitpod.io/from-referrer/)
|
|
135/0 |
MathlibTest/FieldSimp.lean |
1 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
16-15587 16 days ago |
16-15606 16 days ago |
16-85537 16 days |
16041 |
vihdzp author:vihdzp |
feat(SetTheory/Ordinal/Arithmetic): `Ordinal.toNat` |
A simple function sending ordinals less than `ω` to themselves, and anything else to `0`.
---
- [ ] depends on: #17758
[](https://gitpod.io/from-referrer/)
|
t-set-theory
t-logic
awaiting-author
WIP
|
58/0 |
Mathlib/SetTheory/Ordinal/Arithmetic.lean |
1 |
4 |
['github-actions', 'mathlib4-dependent-issues-bot', 'urkud', 'vihdzp'] |
nobody |
15-85706 15 days ago |
15-85708 15 days ago |
54-31491 54 days |
29055 |
vihdzp author:vihdzp |
feat: `Ordinal.toENat` |
We essentially copy the Cardinal/ENat file but make it for ordinals instead. See [Zulip](https://leanprover.zulipchat.com/#narrow/channel/144837-PR-reviews/topic/.2317758.20Ordinal.2EtoENat/near/479768508) for some prior discussion on this PR (particularly, the duplication and how there's no easy way to resolve it.)
---
Moved from #17758.
[](https://gitpod.io/from-referrer/)
|
t-set-theory |
292/0 |
Mathlib.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/SetTheory/Cardinal/ENat.lean,Mathlib/SetTheory/Ordinal/Arithmetic.lean,Mathlib/SetTheory/Ordinal/Basic.lean,Mathlib/SetTheory/Ordinal/ENat.lean |
6 |
1 |
['github-actions'] |
nobody |
15-81744 15 days ago |
16-1134 16 days ago |
16-1156 16 days |
29047 |
grunweg author:grunweg |
chore(1000.yaml): add Fourier's theorem |
Mathlib has some form of it already; while there is space for more advanced versions, let's surface the current progress already.
---
[](https://gitpod.io/from-referrer/)
|
delegated |
5/1 |
docs/1000.yaml |
1 |
4 |
['Ruben-VandeVelde', 'bryangingechen', 'github-actions', 'mathlib-bors'] |
nobody |
15-77855 15 days ago |
15-77855 15 days ago |
0-17788 4 hours |
29033 |
faenuccio author:faenuccio |
feat (???): a linear map is surjective iff its image contains a ball |
---
[](https://gitpod.io/from-referrer/)
|
t-analysis
WIP
|
9/0 |
Mathlib/Analysis/Seminorm.lean |
1 |
1 |
['github-actions'] |
nobody |
15-72668 15 days ago |
16-57270 16 days ago |
0-12 12 seconds |
28889 |
Timeroot author:Timeroot |
Experiment for MulOneClass -> Mul + One together |
Compare with #28702 which uses MulOne together
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
63/55 |
Mathlib/Algebra/Group/Ext.lean,Mathlib/Algebra/Group/Hom/Defs.lean,Mathlib/Algebra/Order/Nonneg/Basic.lean,Mathlib/Analysis/Normed/Group/SemiNormedGrp/Completion.lean,Mathlib/LinearAlgebra/QuadraticForm/Basic.lean,scripts/noshake.json |
6 |
4 |
['Timeroot', 'github-actions', 'leanprover-bot'] |
nobody |
15-71635 15 days ago |
15-71635 15 days ago |
0-0 0 seconds |
28630 |
Antidite author:Antidite |
feat(Archive/Imo): right isosceles configuration in the complex plane |
feat(Archive/Imo): right isosceles configuration in the complex plane
This adds `Archive/Imo/Imo1975Q3.lean`, formalizing a triangle configuration
with points A=0, B=1, C=z and auxiliary points R, P, Q built via complex
rotations and sine-based scale factors.
Main results:
* `angle_and_distance`: ∠QRP = π/2 and dist Q R = dist R P.
* Key identity `QRP_rot90`: (Q z).z − R.z = e^{iπ/2} · ((P z).z − R.z).
Design/Style:
* Minimal imports; module docstring; semantic lemma names; all definitions and
theorems live under the namespace `IMO.TriangleConfig`.
Moves:
- (none)
Deletions:
- (none)
---
[](https://gitpod.io/from-referrer/)
|
IMO
new-contributor
|
196/0 |
Archive.lean,Archive/Imo/Imo1975Q3.lean |
2 |
36 |
['Antidite', 'LLaurance', 'github-actions', 'jsm28'] |
jsm28 assignee:jsm28 |
15-65114 15 days ago |
25-5877 25 days ago |
25-5918 25 days |
25500 |
eric-wieser author:eric-wieser |
feat: delaborators for metadata |
Being able to see these is very important when debugging tactic failures. Probably these could be upstreamed, but I don't think that's a reason not to merge them here first.
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-meta
delegated
awaiting-author
|
75/3 |
Mathlib/Util/Delaborators.lean,Mathlib/Util/PPOptions.lean,MathlibTest/delaborators.lean |
3 |
18 |
['JovanGerb', 'Rob23oba', 'eric-wieser', 'github-actions', 'kmill', 'mathlib-bors', 'plp127'] |
alexjbest assignee:alexjbest |
15-63076 15 days ago |
15-63958 15 days ago |
83-71907 83 days |
27392 |
Paul-Lez author:Paul-Lez |
feat(Tactic/SimpUtils): add simproc finding commands |
This PR adds some commands to allow users to find simprocs/dsimprocs/simp theorems that match on a given pattern.
Thanks to Robin Arnez for telling me about `simprocDeclExt` :)
---
[](https://gitpod.io/from-referrer/)
|
t-meta |
690/0 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/SimpUtils.lean,MathlibTest/SimpUtils.lean |
4 |
9 |
['Paul-Lez', 'eric-wieser', 'github-actions', 'kmill'] |
robertylewis assignee:robertylewis |
15-62212 15 days ago |
38-48951 1 month ago |
40-49618 40 days |
28441 |
euprunin author:euprunin |
chore(GroupTheory/Perm): golf entire `mem_of_formPerm_ne_self` |
---
[](https://gitpod.io/from-referrer/)
|
t-group-theory
awaiting-author
|
2/5 |
Mathlib/GroupTheory/Perm/List.lean |
1 |
2 |
['JonBannon', 'github-actions', 'tb65536'] |
tb65536 assignee:tb65536 |
15-60017 15 days ago |
15-60017 15 days ago |
13-75804 13 days |
28492 |
euprunin author:euprunin |
chore(Data/Finite): golf entire `card_le_of_injective`, `card_le_of_surjective` and `card_sum` |
---
[](https://gitpod.io/from-referrer/)
|
t-data
awaiting-author
|
6/13 |
Mathlib/Data/Finite/Card.lean |
1 |
2 |
['github-actions', 'tb65536'] |
nobody |
15-30804 15 days ago |
15-30804 15 days ago |
13-27739 13 days |
28488 |
euprunin author:euprunin |
chore(SetTheory): golf entire `cast_succ`, `mk_multiset_of_countable` and `iSup_succ` |
---
[](https://gitpod.io/from-referrer/)
|
t-set-theory
awaiting-author
|
6/11 |
Mathlib/SetTheory/Cardinal/Basic.lean,Mathlib/SetTheory/Cardinal/Finsupp.lean,Mathlib/SetTheory/Ordinal/Family.lean |
3 |
5 |
['github-actions', 'vihdzp'] |
nobody |
15-28700 15 days ago |
15-42725 15 days ago |
13-23224 13 days |
28484 |
euprunin author:euprunin |
chore(Data): golf entire `add_one_le_exp_of_nonneg`, `toReal_eq_toReal`, `count_eq_of_nodup`, `smul_mat_cons` and `coe_inj` |
---
[](https://gitpod.io/from-referrer/)
|
t-data |
8/13 |
Mathlib/Combinatorics/Matroid/Minor/Restrict.lean,Mathlib/Data/ENNReal/Real.lean,Mathlib/Data/List/Nodup.lean,Mathlib/LinearAlgebra/Matrix/Notation.lean |
4 |
6 |
['github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
15-19869 15 days ago |
15-19892 15 days ago |
28-34517 28 days |
28316 |
eric-wieser author:eric-wieser |
feat(Tactic/NormNum): better trace nodes |
Comparing the infoview on the first example in the test file
| Before | After |
|---|---|
| | |
In the after version, the extension names are all clickable.
Similar to #21450.
---
[](https://gitpod.io/from-referrer/)
|
t-meta |
136/5 |
Mathlib.lean,Mathlib/Tactic/NormNum/Core.lean,Mathlib/Util/Trace.lean,MathlibTest/norm_num_trace.lean |
4 |
19 |
['JovanGerb', 'eric-wieser', 'github-actions', 'kmill', 'leanprover-bot', 'mathlib-bors', 'plp127'] |
JovanGerb assignee:JovanGerb |
15-15098 15 days ago |
31-42982 1 month ago |
31-42968 31 days |
29072 |
yury-harmonic author:yury-harmonic |
feat({Nat,Int}/ModEq): add lemmas |
---
I'm not sure that I named these lemmas correctly. Suggestions about better names are welcome!
[](https://gitpod.io/from-referrer/)
|
t-data
awaiting-zulip
|
171/15 |
Mathlib/Data/Int/ModEq.lean,Mathlib/Data/Nat/ModEq.lean |
2 |
5 |
['eric-wieser', 'github-actions', 'yury-harmonic'] |
nobody |
15-11121 15 days ago |
15-11121 15 days ago |
0-55232 15 hours |
28669 |
kckennylau author:kckennylau |
chore: clean up some proofs about locally compact valuation |
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
awaiting-author
|
40/25 |
Mathlib/RingTheory/Valuation/Archimedean.lean,Mathlib/Topology/Algebra/Valued/LocallyCompact.lean |
2 |
4 |
['github-actions', 'grunweg', 'kckennylau', 'pechersky'] |
nobody |
15-9593 15 days ago |
15-9636 15 days ago |
9-23828 9 days |
25069 |
erdOne author:erdOne |
feat(EllipticCurve): rational points of singular nodal cubics |
---
[](https://gitpod.io/from-referrer/)
|
t-algebraic-geometry
awaiting-author
|
251/0 |
Mathlib.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Affine/Basic.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Singular/Node.lean |
3 |
13 |
['Multramate', 'acmepjz', 'chrisflav', 'erdOne', 'github-actions', 'grunweg'] |
chrisflav assignee:chrisflav |
15-7882 15 days ago |
15-7882 15 days ago |
100-22151 100 days |
26484 |
peabrainiac author:peabrainiac |
feat(Geometry/Diffeology): basics of diffeological spaces |
Introduces diffeological spaces, smooth maps between them, the D-topology and the standard diffeology on finite-dimensional normed spaces.
---
This PR continues the work from #21969. |
t-differential-geometry |
471/0 |
Mathlib.lean,Mathlib/Geometry/Diffeology/Basic.lean,docs/references.bib |
3 |
10 |
['JovanGerb', 'github-actions', 'grunweg', 'lecopivo', 'peabrainiac'] |
grunweg assignee:grunweg |
15-6544 15 days ago |
77-27760 2 months ago |
77-32509 77 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'] |
joneugster assignee:joneugster |
15-6300 15 days ago |
84-43863 2 months ago |
84-48471 84 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
awaiting-author
|
48/0 |
Mathlib/Tactic/Linter/CommandStart.lean |
1 |
7 |
['adomani', 'github-actions', 'grunweg', 'leanprover-bot'] |
joneugster assignee:joneugster |
15-6152 15 days ago |
15-6274 15 days ago |
66-73556 66 days |
25743 |
robin-carlier author:robin-carlier |
feat(AlgebraicTopology/SimplexCategory/Augmented): monoidal structure on `AugmentedSimplexCategory` |
We construct a monoidal category structure on `AugmentedSimplexCategory`. The tensor products corresponds to ordinal sum. We characterize morphisms out of a tensor product of object in terms of their precomposition with canonical maps `x ⟶ x ⊗ y` and `y ⟶ x ⊗ y` coming from the fact that the unit is an initial object.
When constructing this structure, we found that making `AugmentedSimplexCategory` an abbrev rather than a `def`
worked better.
---
- [x] depends on: #25742
Future work includes using this monoidal structure and Day convolution to define the join monoidal structure on augmented simplicial sets, and also using this category as a way to encode monoidal and monadic bar constructions.
Happy to discuss the fact that I had to make `AugmentedSimplexCategory` an abbrev, I can revert this but this makes the proofs a bit harder (but, I guess, also less abusing some of defeqs?).
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #22768.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/22768* |
t-algebraic-topology
t-category-theory
|
476/114 |
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 |
19 |
['dagurtomas', 'github-actions', 'grunweg', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'robin-carlier'] |
dagurtomas assignee:dagurtomas |
14-84485 14 days ago |
14-84485 14 days ago |
81-62957 81 days |
28474 |
astrainfinita author:astrainfinita |
feat: add `ContinuousSMul` instances for `ℚ≥0` |
---
[](https://gitpod.io/from-referrer/)
|
bench-after-CI
t-algebra
t-topology
awaiting-author
label:t-algebra$ |
14/0 |
Mathlib/Topology/Instances/Rat.lean |
1 |
11 |
['astrainfinita', 'github-actions', 'ocfnash', 'themathqueen'] |
ocfnash assignee:ocfnash |
14-77505 14 days ago |
28-68621 28 days ago |
28-75420 28 days |
27516 |
gaetanserre author:gaetanserre |
feat: add rational approximation lemma for suprema in `unitInterval` |
Add `sSup_eq_iUnion_rat` lemma that provides a rational approximation characterization of suprema in the unit interval. For monotone functions `f : α → I → ℝ`, the lemma establishes that the set of pairs where `a < sSup {x | f e.1 x < e.2}` equals the union over all rationals `q ∈ I` with `q > a` of the sets `{e | f e.1 q < e.2}`.
---
[](https://gitpod.io/from-referrer/)
|
t-topology |
44/0 |
Mathlib/MeasureTheory/Constructions/UnitInterval.lean,Mathlib/Topology/UnitInterval.lean |
2 |
6 |
['gaetanserre', 'github-actions', 'mathlib4-merge-conflict-bot', 'ocfnash'] |
ocfnash assignee:ocfnash |
14-69835 14 days ago |
19-71554 19 days ago |
45-62555 45 days |
27468 |
IvanRenison author:IvanRenison |
feat(Combinatorics/SimpleGraph): add theorem `SimpleGraph.Connected.diff_dist_adj` |
This contribution was created as part of the Utrecht Summerschool "Formalizing Mathematics in Lean" in July 2025.
---
[](https://gitpod.io/from-referrer/)
|
t-combinatorics |
8/0 |
Mathlib/Combinatorics/SimpleGraph/Metric.lean |
1 |
5 |
['b-mehta', 'github-actions', 'vlad902'] |
awainverse assignee:awainverse |
14-67839 14 days ago |
49-78975 1 month ago |
49-79070 49 days |
27461 |
IvanRenison author:IvanRenison |
feat(Combinatorics/SimpleGraph/Paths): add lemma `SimpleGraph.Walk.IsPath.mem_support_iff_exists_append` |
This contribution was created as part of the Utrecht Summerschool "Formalizing Mathematics in Lean" in July 2025.
---
[](https://gitpod.io/from-referrer/)
|
t-combinatorics |
14/0 |
Mathlib/Combinatorics/SimpleGraph/Paths.lean |
1 |
3 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
awainverse assignee:awainverse |
14-66992 14 days ago |
14-68114 14 days ago |
44-82785 44 days |
26913 |
Paul-Lez author:Paul-Lez |
feat(NumberTheory/{*}): add a few lemmas about number field and cyclotomic extensions |
The motivation for this PR is that the main statement in [this PR](https://github.com/google-deepmind/formal-conjectures/pull/297) shouldn't need to assume `p` has type `PNat` for the instances to work.
This is still WIP as I need to clean up (currently waiting on the build!)
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-number-theory
awaiting-CI
WIP
label:t-algebra$ |
52/0 |
Mathlib/NumberTheory/ClassNumber/Temporary.lean,Mathlib/NumberTheory/Cyclotomic/Basic.lean,Mathlib/NumberTheory/Cyclotomic/Embeddings.lean,Mathlib/NumberTheory/NumberField/InfinitePlace/TotallyRealComplex.lean |
4 |
1 |
['github-actions'] |
nobody |
14-52964 14 days ago |
14-53090 14 days ago |
0-28 28 seconds |
27433 |
YaelDillies author:YaelDillies |
refactor: make `⇑e⁻¹ = e.symm` simp |
From BrauerGroup and ClassFieldTheory
---
[](https://gitpod.io/from-referrer/)
|
|
217/256 |
Mathlib/Algebra/Algebra/Equiv.lean,Mathlib/Algebra/Group/End.lean,Mathlib/Algebra/Module/Equiv/Basic.lean,Mathlib/Algebra/Order/Rearrangement.lean,Mathlib/Data/Fintype/Perm.lean,Mathlib/FieldTheory/KrullTopology.lean,Mathlib/GroupTheory/Perm/Basic.lean,Mathlib/GroupTheory/Perm/Centralizer.lean,Mathlib/GroupTheory/Perm/Cycle/Basic.lean,Mathlib/GroupTheory/Perm/Cycle/Factors.lean,Mathlib/GroupTheory/Perm/Finite.lean,Mathlib/GroupTheory/Perm/Sign.lean,Mathlib/GroupTheory/Perm/Support.lean,Mathlib/GroupTheory/SpecificGroups/Alternating.lean,Mathlib/LinearAlgebra/Matrix/Determinant/Basic.lean,Mathlib/Logic/Equiv/Set.lean |
16 |
3 |
['eric-wieser', 'github-actions'] |
dwrensha assignee:dwrensha |
14-34937 14 days ago |
26-75067 26 days ago |
27-20035 27 days |
27672 |
b-reinke author:b-reinke |
feat(GroupTheory/FreeGroup): add definition of cyclically reduced words |
This PR adds the definition of cyclically reduced words for free groups. It is a part of a series of PR on the theory of cyclically reduced words.
Upstreamed from the [EquationalTheories](https://github.com/teorth/equational_theories) project.
- [ ] depends on: #25966
---
[](https://gitpod.io/from-referrer/)
|
t-group-theory |
72/0 |
Mathlib.lean,Mathlib/GroupTheory/FreeGroup/CyclicallyReduced.lean |
2 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
tb65536 assignee:tb65536 |
14-34936 14 days ago |
29-70102 29 days ago |
29-73233 29 days |
28560 |
euprunin author:euprunin |
chore(Combinatorics/Quiver): golf entire `lift_spec` using `rfl` |
---
Show trace profiling of lift_spec : <10 ms before, <10 ms after 🎉
### Trace profiling of `lift_spec` before PR 28560
```diff
diff --git a/Mathlib/Combinatorics/Quiver/Symmetric.lean b/Mathlib/Combinatorics/Quiver/Symmetric.lean
index 33e371b283..76a3371b36 100644
--- a/Mathlib/Combinatorics/Quiver/Symmetric.lean
+++ b/Mathlib/Combinatorics/Quiver/Symmetric.lean
@@ -164,6 +164,7 @@ def lift [HasReverse V'] (φ : Prefunctor V V') :
| Sum.inl g => φ.map g
| Sum.inr g => reverse (φ.map g)
+set_option trace.profiler true in
theorem lift_spec [HasReverse V'] (φ : Prefunctor V V') :
Symmetrify.of.comp (Symmetrify.lift φ) = φ := by
fapply Prefunctor.ext
```
```
✔ [147/147] Built Mathlib.Combinatorics.Quiver.Symmetric (1.3s)
Build completed successfully (147 jobs).
```
### Trace profiling of `lift_spec` after PR 28560
```diff
diff --git a/Mathlib/Combinatorics/Quiver/Symmetric.lean b/Mathlib/Combinatorics/Quiver/Symmetric.lean
index 33e371b283..3adf874946 100644
--- a/Mathlib/Combinatorics/Quiver/Symmetric.lean
+++ b/Mathlib/Combinatorics/Quiver/Symmetric.lean
@@ -164,13 +164,10 @@ def lift [HasReverse V'] (φ : Prefunctor V V') :
| Sum.inl g => φ.map g
| Sum.inr g => reverse (φ.map g)
+set_option trace.profiler true in
theorem lift_spec [HasReverse V'] (φ : Prefunctor V V') :
Symmetrify.of.comp (Symmetrify.lift φ) = φ := by
- fapply Prefunctor.ext
- · rintro X
- rfl
- · rintro X Y f
- rfl
+ tauto
theorem lift_reverse [h : HasInvolutiveReverse V']
(φ : Prefunctor V V') {X Y : Symmetrify V} (f : X ⟶ Y) :
```
```
✔ [147/147] Built Mathlib.Combinatorics.Quiver.Symmetric (1.2s)
Build completed successfully (147 jobs).
```
---
[](https://gitpod.io/from-referrer/)
|
t-combinatorics |
2/6 |
Mathlib/Combinatorics/Quiver/Symmetric.lean |
1 |
1 |
['github-actions'] |
awainverse assignee:awainverse |
14-34930 14 days ago |
26-63185 26 days ago |
26-63232 26 days |
28574 |
euprunin author:euprunin |
chore(Topology/Category): golf entire `finiteCoproduct.ι_desc_apply`, `piIsoPi_hom_apply`, `prodIsoProd_hom_apply` and `pullbackIsoProdSubtype_hom_apply` using `tauto` and `rfl` |
---
Show trace profiling of finiteCoproduct.ι_desc_apply : 15 ms before, 25 ms after
### Trace profiling of `finiteCoproduct.ι_desc_apply` before PR 28574
```diff
diff --git a/Mathlib/Topology/Category/CompHausLike/Limits.lean b/Mathlib/Topology/Category/CompHausLike/Limits.lean
index 493c277fec..216c5888f2 100644
--- a/Mathlib/Topology/Category/CompHausLike/Limits.lean
+++ b/Mathlib/Topology/Category/CompHausLike/Limits.lean
@@ -109,6 +109,7 @@ lemma finiteCoproduct.ι_injective (a : α) : Function.Injective (finiteCoproduc
lemma finiteCoproduct.ι_jointly_surjective (R : finiteCoproduct X) :
∃ (a : α) (r : X a), R = finiteCoproduct.ι X a r := ⟨R.fst, R.snd, rfl⟩
+set_option trace.profiler true in
lemma finiteCoproduct.ι_desc_apply {B : CompHausLike P} {π : (a : α) → X a ⟶ B} (a : α) :
∀ x, finiteCoproduct.desc X π (finiteCoproduct.ι X a x) = π a x := by
intro x
```
```
ℹ [985/985] Built Mathlib.Topology.Category.CompHausLike.Limits (1.9s)
info: Mathlib/Topology/Category/CompHausLike/Limits.lean:113:0: [Elab.command] [0.011940] theorem ι_desc_apply {B : CompHausLike P} {π : (a : α) → X a ⟶ B} (a : α) :
∀ x, finiteCoproduct.desc X π (finiteCoproduct.ι X a x) = π a x :=
by
intro x
change (ι X a ≫ desc X π) _ = _
simp only [ι_desc]
[Elab.definition.header] [0.011212] CompHausLike.finiteCoproduct.ι_desc_apply
[Elab.step] [0.010053] expected type: Sort ?u.7530, term
∀ x, finiteCoproduct.desc X π (finiteCoproduct.ι X a x) = π a x
info: Mathlib/Topology/Category/CompHausLike/Limits.lean:113:0: [Elab.command] [0.012175] theorem finiteCoproduct.ι_desc_apply {B : CompHausLike P} {π : (a : α) → X a ⟶ B} (a : α) :
∀ x, finiteCoproduct.desc X π (finiteCoproduct.ι X a x) = π a x :=
by
intro x
change (ι X a ≫ desc X π) _ = _
simp only [ι_desc]
info: Mathlib/Topology/Category/CompHausLike/Limits.lean:113:0: [Elab.command] [0.012211] lemma finiteCoproduct.ι_desc_apply {B : CompHausLike P} {π : (a : α) → X a ⟶ B} (a : α) :
∀ x, finiteCoproduct.desc X π (finiteCoproduct.ι X a x) = π a x :=
by
intro x
change (ι X a ≫ desc X π) _ = _
simp only [ι_desc]
info: Mathlib/Topology/Category/CompHausLike/Limits.lean:113:0: [Elab.async] [0.015416] elaborating proof of CompHausLike.finiteCoproduct.ι_desc_apply
[Elab.definition.value] [0.014903] CompHausLike.finiteCoproduct.ι_desc_apply
[Elab.step] [0.014576]
intro x
change (ι X a ≫ desc X π) _ = _
simp only [ι_desc]
[Elab.step] [0.014564]
intro x
change (ι X a ≫ desc X π) _ = _
simp only [ι_desc]
[Elab.step] [0.011699] change (ι X a ≫ desc X π) _ = _
Build completed successfully (985 jobs).
```
### Trace profiling of `finiteCoproduct.ι_desc_apply` after PR 28574
```diff
diff --git a/Mathlib/Topology/Category/CompHausLike/Limits.lean b/Mathlib/Topology/Category/CompHausLike/Limits.lean
index 493c277fec..b70ed614b6 100644
--- a/Mathlib/Topology/Category/CompHausLike/Limits.lean
+++ b/Mathlib/Topology/Category/CompHausLike/Limits.lean
@@ -109,11 +109,10 @@ lemma finiteCoproduct.ι_injective (a : α) : Function.Injective (finiteCoproduc
lemma finiteCoproduct.ι_jointly_surjective (R : finiteCoproduct X) :
∃ (a : α) (r : X a), R = finiteCoproduct.ι X a r := ⟨R.fst, R.snd, rfl⟩
+set_option trace.profiler true in
lemma finiteCoproduct.ι_desc_apply {B : CompHausLike P} {π : (a : α) → X a ⟶ B} (a : α) :
∀ x, finiteCoproduct.desc X π (finiteCoproduct.ι X a x) = π a x := by
- intro x
- change (ι X a ≫ desc X π) _ = _
- simp only [ι_desc]
+ tauto
instance : HasCoproduct X where
exists_colimit := ⟨finiteCoproduct.cofan X, finiteCoproduct.isColimit X⟩
diff --git a/Mathlib/Topology/Category/TopCat/Limits/Products.lean b/Mathlib/Topology/Category/TopCat/Limits/Products.lean
index 0b74c2f6ee..353896fce8 100644
--- a/Mathlib/Topology/Category/TopCat/Limits/Products.lean
+++ b/Mathlib/Topology/Category/TopCat/Limits/Products.lean
@@ -62,9 +62,7 @@ theorem piIsoPi_inv_π_apply {ι : Type v} (α : ι → TopCat.{max v u}) (i :
theorem piIsoPi_hom_apply {ι : Type v} (α : ι → TopCat.{max v u}) (i : ι)
(x : (∏ᶜ α : TopCat.{max v u})) : (piIsoPi α).hom x i = (Pi.π α i :) x := by
- have := piIsoPi_inv_π α i
- rw [Iso.inv_comp_eq] at this
- exact ConcreteCategory.congr_hom this x
+ tauto
/-- The inclusion to the coproduct as a bundled continuous map. -/
abbrev sigmaι {ι : Type v} (α : ι → TopCat.{max v u}) (i : ι) : α i ⟶ TopCat.of (Σ i, α i) := by
@@ -165,9 +163,7 @@ theorem prodIsoProd_hom_snd (X Y : TopCat.{u}) :
theorem prodIsoProd_hom_apply {X Y : TopCat.{u}} (x : ↑(X ⨯ Y)) :
(prodIsoProd X Y).hom x = ((Limits.prod.fst : X ⨯ Y ⟶ _) x,
(Limits.prod.snd : X ⨯ Y ⟶ _) x) := by
- ext
- · exact ConcreteCategory.congr_hom (prodIsoProd_hom_fst X Y) x
- · exact ConcreteCategory.congr_hom (prodIsoProd_hom_snd X Y) x
+ tauto
@[reassoc (attr := simp), elementwise]
theorem prodIsoProd_inv_fst (X Y : TopCat.{u}) :
diff --git a/Mathlib/Topology/Category/TopCat/Limits/Pullbacks.lean b/Mathlib/Topology/Category/TopCat/Limits/Pullbacks.lean
index 66049170b3..68b42db21b 100644
--- a/Mathlib/Topology/Category/TopCat/Limits/Pullbacks.lean
+++ b/Mathlib/Topology/Category/TopCat/Limits/Pullbacks.lean
@@ -110,9 +110,7 @@ theorem pullbackIsoProdSubtype_hom_apply {f : X ⟶ Z} {g : Y ⟶ Z}
(pullbackIsoProdSubtype f g).hom x =
⟨⟨pullback.fst f g x, pullback.snd f g x⟩, by
simpa using CategoryTheory.congr_fun pullback.condition x⟩ := by
- apply Subtype.ext; apply Prod.ext
- exacts [ConcreteCategory.congr_hom (pullbackIsoProdSubtype_hom_fst f g) x,
- ConcreteCategory.congr_hom (pullbackIsoProdSubtype_hom_snd f g) x]
+ tauto
theorem pullback_topology {X Y Z : TopCat.{u}} (f : X ⟶ Z) (g : Y ⟶ Z) :
(pullback f g).str =
```
```
✔ [982/985] Built Mathlib.Topology.Category.TopCat.Limits.Products (2.7s)
✔ [983/985] Built Mathlib.Topology.Category.TopCat.Limits.Pullbacks (2.4s)
✔ [984/985] Built Mathlib.CategoryTheory.Extensive (4.3s)
ℹ [985/985] Built Mathlib.Topology.Category.CompHausLike.Limits (3.0s)
info: Mathlib/Topology/Category/CompHausLike/Limits.lean:113:0: [Elab.command] [0.033044] theorem ι_desc_apply {B : CompHausLike P} {π : (a : α) → X a ⟶ B} (a : α) :
∀ x, finiteCoproduct.desc X π (finiteCoproduct.ι X a x) = π a x := by tauto
[Elab.definition.header] [0.031659] CompHausLike.finiteCoproduct.ι_desc_apply
[Elab.step] [0.030394] expected type: Sort ?u.7530, term
∀ x, finiteCoproduct.desc X π (finiteCoproduct.ι X a x) = π a x
[Elab.step] [0.030250] expected type: Sort ?u.7534, term
finiteCoproduct.desc X π (finiteCoproduct.ι X a x) = π a x
[Elab.step] [0.030242] expected type: Sort ?u.7534, term
binrel% Eq✝ (finiteCoproduct.desc X π (finiteCoproduct.ι X a x)) (π a x)
[Elab.step] [0.025815] expected type: , term
finiteCoproduct.desc X π (finiteCoproduct.ι X a x)
[Elab.step] [0.010204] expected type: (fun X ↦ ↑X.toTop) (finiteCoproduct X), term
(finiteCoproduct.ι X a x)
[Elab.step] [0.010186] expected type: (fun X ↦ ↑X.toTop) (finiteCoproduct X), term
finiteCoproduct.ι X a x
info: Mathlib/Topology/Category/CompHausLike/Limits.lean:113:0: [Elab.command] [0.033536] theorem finiteCoproduct.ι_desc_apply {B : CompHausLike P} {π : (a : α) → X a ⟶ B} (a : α) :
∀ x, finiteCoproduct.desc X π (finiteCoproduct.ι X a x) = π a x := by tauto
info: Mathlib/Topology/Category/CompHausLike/Limits.lean:113:0: [Elab.command] [0.033652] lemma finiteCoproduct.ι_desc_apply {B : CompHausLike P} {π : (a : α) → X a ⟶ B} (a : α) :
∀ x, finiteCoproduct.desc X π (finiteCoproduct.ι X a x) = π a x := by tauto
info: Mathlib/Topology/Category/CompHausLike/Limits.lean:113:0: [Elab.async] [0.025323] elaborating proof of CompHausLike.finiteCoproduct.ι_desc_apply
[Elab.definition.value] [0.024806] CompHausLike.finiteCoproduct.ι_desc_apply
[Elab.step] [0.024330] tauto
[Elab.step] [0.024317] tauto
[Elab.step] [0.024304] tauto
Build completed successfully (985 jobs).
```
---
[](https://gitpod.io/from-referrer/)
|
t-topology |
4/15 |
Mathlib/Topology/Category/CompHausLike/Limits.lean,Mathlib/Topology/Category/TopCat/Limits/Products.lean,Mathlib/Topology/Category/TopCat/Limits/Pullbacks.lean |
3 |
1 |
['github-actions'] |
ADedecker assignee:ADedecker |
14-34929 14 days ago |
26-62547 26 days ago |
26-62587 26 days |
28699 |
chrisflav author:chrisflav |
feat(RingTheory/Cotangent): cotangent of composition with localization away from an element |
Let `R → S → T` be algebras such that `T` is the localization of `S` away from one
element, where `S` is generated over `R` by `P : R[X] → S` with kernel `I` and
`Q : S[Y] → T` is the canonical `S`-presentation of `T` with kernel `K`.
Denote by `J` the kernel of the composition `R[X,Y] → T`.
We deduce `J/J² ≃ₗ[T] T ⊗[S] (I/I²) × K/K²` from the Jacobi Zariski sequence.
From Pi1.
---
- [x] depends on: #28697
The import increase is expected: This file was PRed in two steps and only the second one depends on more imports.
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
large-import
|
147/4 |
Mathlib/RingTheory/Extension/Cotangent/LocalizationAway.lean,Mathlib/RingTheory/Extension/Generators.lean,Mathlib/RingTheory/Extension/Presentation/Basic.lean,Mathlib/RingTheory/Smooth/StandardSmoothCotangent.lean |
4 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
mattrobball assignee:mattrobball |
14-34927 14 days ago |
22-76725 22 days ago |
22-78138 22 days |
28772 |
chrisflav author:chrisflav |
feat(RingTheory/IsTensorProduct): add `IsPushout.cancelBaseChange` |
This is a cancel-on-the-left version of `AlgebraTensorModule.cancelBaseChange`.
---
[](https://gitpod.io/from-referrer/) |
t-ring-theory |
49/0 |
Mathlib/RingTheory/IsTensorProduct.lean |
1 |
1 |
['github-actions'] |
erdOne assignee:erdOne |
14-34923 14 days ago |
22-7749 22 days ago |
22-7730 22 days |
29089 |
hrmacbeth author:hrmacbeth |
feat: field tactic |
This PR creates a `field` tactic, i.e. an analogue of `ring` but for fields -- a finishing tactic for equality goals in fields. It is basically `field_simp; ring1`, with a few tweaks for better error reporting!
We could have done this at any point in the last five years, but since `field_simp` is more performant as of #28658, now seems like a good time.
I propose that `field` be preferred to terminal `field_simp`/`field_simp; ring` from now on. I'll follow up with a PR ([preview](https://github.com/leanprover-community/mathlib4/commit/44c0136fb8650f57416733d0b336c60b338f3d99)) making this change widely across the library. In the current PR I also rewrote the docstrings of `field_simp` and friends to nudge users in this direction.
Closes #4837
---
[](https://gitpod.io/from-referrer/)
|
t-meta |
315/24 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Field.lean,Mathlib/Tactic/FieldSimp.lean,MathlibTest/FieldSimp.lean |
5 |
31 |
['github-actions', 'grunweg', 'hrmacbeth'] |
grunweg assignee:grunweg |
14-15027 14 days ago |
14-41260 14 days ago |
14-42883 14 days |
28486 |
euprunin author:euprunin |
chore(Order): golf entire `map_covBy`, `covBy_of_apply`, `map_wcovBy`, `wcovBy_of_apply`, `ne_bot_of_ne_top'`, `insert_Icc_left_eq_Icc_pred` and `insert_Icc_right_eq_Icc_succ` |
---
[](https://gitpod.io/from-referrer/)
|
t-order
awaiting-author
|
14/24 |
Mathlib/Order/Cover.lean,Mathlib/Order/Disjoint.lean,Mathlib/Order/Interval/Set/SuccPred.lean |
3 |
6 |
['YaelDillies', 'bryangingechen', 'github-actions', 'mathlib4-merge-conflict-bot'] |
bryangingechen assignee:bryangingechen |
14-12147 14 days ago |
14-12147 14 days ago |
14-50468 14 days |
26455 |
ScottCarnahan author:ScottCarnahan |
WIP - feat (LinearAlgebra/RootSystem): API for CartanMatrix |
Some attempts at working out good ways to eliminate bad Cartan matrices.
Very much WIP
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
WIP
label:t-algebra$ |
815/26 |
Mathlib/Algebra/Group/Action/Faithful.lean,Mathlib/LinearAlgebra/LinearIndependent/Basic.lean,Mathlib/LinearAlgebra/RootSystem/Base.lean,Mathlib/LinearAlgebra/RootSystem/CartanMatrix.lean,Mathlib/LinearAlgebra/RootSystem/Finite/CanonicalBilinear.lean,Mathlib/LinearAlgebra/RootSystem/Finite/Lemmas.lean,Mathlib/LinearAlgebra/RootSystem/GeckConstruction/Relations.lean,Mathlib/LinearAlgebra/RootSystem/IsValuedIn.lean,Mathlib/LinearAlgebra/RootSystem/RootPositive.lean |
9 |
7 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-merge-conflict-bot'] |
nobody |
14-10680 14 days ago |
14-10698 14 days ago |
0-17731 4 hours |
29014 |
ShreckYe author:ShreckYe |
feat(Data/List/Scan): some theorems that relate `scanl` with `foldl` |
I am not sure which is the best form of `getElem_scanl_eq_foldl_take` here, so I added several alternative forms. Feel free to remove any of them if necessary. |
t-data |
35/0 |
Mathlib/Data/List/Scan.lean |
1 |
9 |
['ShreckYe', 'github-actions', 'themathqueen', 'vlad902'] |
nobody |
14-9765 14 days ago |
17-5012 17 days ago |
17-5057 17 days |
28891 |
joelriou author:joelriou |
feat(Analysis/Convex): functoriality of the standard simplex |
When `f : X → Y` is a map between finite types, and `S` is an ordered semiring, we define the maps `stdSimplex.map f : stdSimplex S X → stdSimplex S Y`. In the case `S := ℝ`, we show that these maps are continuous. In a future PR #28893, the definition of the topological simplex in `AlgebraicTopology` shall be refactored.
---
- [x] depends on: #28869
[](https://gitpod.io/from-referrer/)
|
t-convex-geometry |
192/1 |
Mathlib.lean,Mathlib/Analysis/Convex/StdSimplex.lean,Mathlib/LinearAlgebra/Finsupp/Pi.lean,Mathlib/Topology/Algebra/Monoid/FunOnFinite.lean |
4 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
13-66609 13 days ago |
13-66609 13 days ago |
13-67799 13 days |
29145 |
JovanGerb author:JovanGerb |
chore: use `to_additive` in more places |
This PR addresses some comments about `to_additive` not working, by making it work more.
---
[](https://gitpod.io/from-referrer/)
|
|
61/177 |
Mathlib/Algebra/Group/End.lean,Mathlib/Algebra/Order/BigOperators/Group/LocallyFinite.lean,Mathlib/Combinatorics/Additive/DoublingConst.lean,Mathlib/Data/ZMod/Aut.lean,Mathlib/Topology/Algebra/InfiniteSum/Module.lean |
5 |
3 |
['JovanGerb', 'github-actions'] |
nobody |
13-39655 13 days ago |
13-69594 13 days ago |
13-69575 13 days |
25899 |
pfaffelh author:pfaffelh |
feat(Topology/Compactness/CompactSystem): introduce compact Systems |
A compact system is a set systems with the property that, whenever a countable intersections of sets in the set system is empty, there is a finite subset of sets with empty intersection. These are needed e.g. in measure theory if one wants to show sigma-additivity of a set function on a ring.
* Main result: The set of sets which are either compact and closed, or `univ`, is a compact system.
* Introduce `Dissipate s x := ⋂ y ≤ x, s y` (Data/Set/Dissipate), which is parallel to Data/Set/Accumulate.
Co-authored-by: Rémy Degenne remydegenne@gmail.com
---
*This PR continues the work from #24541.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/24541* |
t-topology |
453/1 |
Mathlib.lean,Mathlib/Data/Set/Accumulate.lean,Mathlib/Data/Set/Dissipate.lean,Mathlib/MeasureTheory/PiSystem.lean,Mathlib/Topology/Compactness/CompactSystem.lean |
5 |
14 |
['github-actions', 'pfaffelh', 'sgouezel'] |
PatrickMassot assignee:PatrickMassot |
13-34915 13 days ago |
23-51616 23 days ago |
64-62202 64 days |
25902 |
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.
---
*This PR continues the work from #22714.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/22714* |
large-import
t-measure-probability
|
260/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 |
5 |
1 |
['github-actions'] |
kex-y assignee:kex-y |
13-34914 13 days ago |
25-45390 25 days ago |
25-55583 25 days |
28390 |
euprunin author:euprunin |
chore(Analysis/LocallyConvex): golf entire `polar_weak_closed` |
---
[](https://gitpod.io/from-referrer/)
|
t-analysis
awaiting-author
|
1/4 |
Mathlib/Analysis/LocallyConvex/Polar.lean |
1 |
2 |
['JonBannon', 'github-actions', 'j-loreaux'] |
j-loreaux assignee:j-loreaux |
13-30758 13 days ago |
13-30758 13 days ago |
16-76176 16 days |
28343 |
RemyDegenne author:RemyDegenne |
feat(Probability): Fernique's theorem for distributions that are invariant by rotation |
Let `μ` be a finite measure on a second-countable normed space `E` such that the product measure `μ.prod μ` on `E × E` is invariant by rotation of angle `-π/4`.
Then there exists a constant `C > 0` such that the function `x ↦ exp (C * ‖x‖ ^ 2)` is integrable with respect to `μ`.
The main application of this theorem will be for Gaussian measures.
---
The PR is large, but is basically one big proof, so I don't think I can cut it at a meaningful place.
- [x] depends on: #28342
[](https://gitpod.io/from-referrer/)
|
t-measure-probability |
617/0 |
Mathlib.lean,Mathlib/Data/Real/Sqrt.lean,Mathlib/Probability/Distributions/Fernique.lean,docs/references.bib |
4 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
kex-y assignee:kex-y |
13-10485 13 days ago |
25-15480 25 days ago |
25-22756 25 days |
26843 |
vasnesterov author:vasnesterov |
feat(Tactic/Simproc): nested quantifiers in `existsAndEq` |
Generalize the `existsAndEq` simproc to nested existential quantifiers.
For example `∃ a, p a ∧ ∃ b, a = f b ∧ q b` now simplifies to `∃ b, p (f b) ∧ q b`.
---
[](https://gitpod.io/from-referrer/)
This PR continues the work from #23365.
Original PR: https://github.com/leanprover-community/mathlib4/pull/23365 |
migrated-from-branch
large-import
t-meta
|
457/77 |
Mathlib/Combinatorics/SimpleGraph/Maps.lean,Mathlib/Data/List/ProdSigma.lean,Mathlib/Tactic/Simproc/ExistsAndEq.lean,MathlibTest/Simproc/ExistsAndEq.lean |
4 |
15 |
['JovanGerb', 'github-actions', 'grunweg', 'leanprover-bot', 'leanprover-community-bot-assistant', 'leanprover-community-mathlib4-bot', 'mathlib4-merge-conflict-bot', 'vasnesterov'] |
kmill assignee:kmill |
12-80923 12 days ago |
13-48315 13 days ago |
67-65853 67 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
awaiting-author
|
358/0 |
Mathlib.lean,Mathlib/MeasureTheory/VectorMeasure/Variation/Defs.lean |
2 |
32 |
['EtienneC30', 'github-actions', 'yoh-tanimoto'] |
EtienneC30 assignee:EtienneC30 |
12-74158 12 days ago |
43-67278 1 month ago |
42-9361 42 days |
28885 |
wwylele author:wwylele |
feat(Algebra): Gauss summation for integers |
The `Nat` version `Finset.sum_range_id` is often awkward to use in linear transformation due to Nat's truncated sub (the `n = 0` case already deviates from the typical meaning of the formula). Add an integer version so one can easily use this with arbitrary starting and ending point, and slide/scale it freely as they need.
Not sure if this is the best home for these theorems. I placed there in the same file as `Finset.sum_Ico_add_eq_sum_Ico_add_one`'s
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebra
label:t-algebra$ |
24/2 |
Mathlib/Algebra/BigOperators/Intervals.lean,Mathlib/Algebra/Order/BigOperators/Group/LocallyFinite.lean |
2 |
1 |
['github-actions'] |
nobody |
12-70897 12 days ago |
12-70897 12 days ago |
0-0 0 seconds |
28676 |
sun123zxy author:sun123zxy |
feat(NumberTheory/ArithmeticFunction): wrap `Nat.totient` as an `ArithmeticFunction` |
This wraps the Euler's totient function `Nat.totient` into a new `ArithmeticFunction` `ϕ`, with some basic identities such as `ϕ * ζ = id` and `μ * id = ϕ.`
---
We use the notation `ϕ` to distinguish from `Nat.totient`'s notation `φ`, however this might be controversial. Suggestions are welcome!
[](https://gitpod.io/from-referrer/)
|
large-import
new-contributor
t-number-theory
|
49/3 |
Mathlib/NumberTheory/ArithmeticFunction.lean |
1 |
10 |
['MichaelStollBayreuth', 'b-mehta', 'eric-wieser', 'github-actions', 'sun123zxy'] |
MichaelStollBayreuth assignee:MichaelStollBayreuth |
12-57237 12 days ago |
24-22081 24 days ago |
24-23049 24 days |
29186 |
winstonyin author:winstonyin |
feat: IsIntegralCurve for solutions to ODEs |
I define `IsIntegralCurve` etc. for solutions to ODEs on vector spaces. The translation and scaling lemmas are also included. This parallels `IsMIntegralCurve` etc. for manifolds.
Moved from #26534.
- [x] depends on: #26563
---
[](https://gitpod.io/from-referrer/)
|
t-dynamics
t-analysis
t-differential-geometry
|
298/0 |
Mathlib.lean,Mathlib/Analysis/ODE/Basic.lean,Mathlib/Analysis/ODE/Transform.lean |
3 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
12-54666 12 days ago |
12-54756 12 days ago |
12-54898 12 days |
28279 |
Equilibris author:Equilibris |
feat: univ generic W |
A simple change making `W.ind`'s motive universe generic.
---
A theorem `w_ind_eq` will now be needed, but this will depend on getting `dcongr_heq` merged, and hence I will do this in a separate PR.
[](https://gitpod.io/from-referrer/)
|
t-data
new-contributor
|
16/21 |
Mathlib/Data/PFunctor/Multivariate/W.lean |
1 |
8 |
['Equilibris', 'alexkeizer', 'github-actions'] |
nobody |
12-52904 12 days ago |
32-14170 1 month ago |
0-0 0 seconds |
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
|
7/5 |
Mathlib/Data/Real/Sqrt.lean |
1 |
5 |
['MichaelStollBayreuth', 'github-actions', 'j-loreaux', 'leanprover-bot'] |
ericrbg assignee:ericrbg |
12-49055 12 days ago |
12-53771 12 days ago |
81-80367 81 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
t-analysis
|
142/2 |
Mathlib.lean,Mathlib/Analysis/InnerProductSpace/GramMatrix.lean,Mathlib/MeasureTheory/Function/L2Space.lean |
3 |
38 |
['EtienneC30', 'eric-wieser', 'github-actions', 'pfaffelh'] |
hrmacbeth assignee:hrmacbeth |
12-34893 12 days ago |
23-51685 23 days ago |
66-73694 66 days |
28296 |
strihanje01 author:strihanje01 |
feat(Combinatorics/Additive/VerySmallDoubling): Hamidoune's Freiman-Kneser theorem for nonabelian groups |
add noncommutative Freiman-Kneser theorem for doubling less than 2-\epsilon
---
[](https://gitpod.io/from-referrer/)
|
large-import
new-contributor
t-combinatorics
|
339/3 |
Mathlib/Combinatorics/Additive/VerySmallDoubling.lean |
1 |
14 |
['YaelDillies', 'github-actions', 'strihanje01'] |
awainverse assignee:awainverse |
12-34891 12 days ago |
22-78145 22 days ago |
24-54992 24 days |
28555 |
YaelDillies author:YaelDillies |
feat: pullback along an epi preserved under pullbacks is faithful |
From Toric
---
[](https://gitpod.io/from-referrer/)
|
toric
large-import
t-category-theory
|
39/2 |
Mathlib/CategoryTheory/Comma/Over/Basic.lean,Mathlib/CategoryTheory/Comma/Over/Pullback.lean |
2 |
1 |
['github-actions'] |
kim-em assignee:kim-em |
12-34889 12 days ago |
26-64375 26 days ago |
26-64632 26 days |
28691 |
or4nge19 author:or4nge19 |
feat(Probability/Invariance):Reversibility/DetailedBalance |
Add reversibility (detailed balance) for Markov kernels and show it implies invariance
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-measure-probability
|
19/1 |
Mathlib/Probability/Kernel/Invariance.lean |
1 |
11 |
['DavidLedvinka', 'github-actions', 'or4nge19'] |
sgouezel assignee:sgouezel |
12-34888 12 days ago |
20-13715 20 days ago |
23-60672 23 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
|
114/23 |
Mathlib/Algebra/Category/MonCat/Adjunctions.lean,Mathlib/Data/Finsupp/Option.lean |
2 |
15 |
['BoltonBailey', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
eric-wieser assignee:eric-wieser |
12-14543 12 days ago |
12-19589 12 days ago |
76-76474 76 days |
26841 |
xroblot author:xroblot |
feat(FieldTheory/IsGalois): map induced by the restriction to a subfield |
For `E/L` a field extension and `K` a subfield of `E`, we define the map `(E ≃ₐ[L] E) →* (K ≃ₐ[F] K)` induced by the restriction to `K` (with `F` a subfield of `K` and `L` such that `K/F` is normal) and study when it is injective and surjective.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
65/0 |
Mathlib/FieldTheory/Galois/Basic.lean |
1 |
7 |
['github-actions', 'tb65536', 'xroblot'] |
Vierkantor assignee:Vierkantor |
12-4198 12 days ago |
68-9843 2 months ago |
68-9887 68 days |
27843 |
JovanGerb author:JovanGerb |
chore(Algebra/Order/Sub/Defs): `@[gcongr low]` for `tsub_le_tsub` |
This PR explicitly lowers the `gcongr` priority of `tsub_le_tsub`. It also golfs some proofs using this `gcongr` lemma
---
[](https://gitpod.io/from-referrer/)
|
t-data |
33/36 |
Mathlib/Algebra/Order/Archimedean/Basic.lean,Mathlib/Algebra/Order/Sub/Defs.lean,Mathlib/Algebra/Polynomial/Derivative.lean,Mathlib/AlgebraicGeometry/EllipticCurve/DivisionPolynomial/Degree.lean,Mathlib/Analysis/Asymptotics/Lemmas.lean,Mathlib/Analysis/Complex/UpperHalfPlane/Metric.lean,Mathlib/Combinatorics/Hall/Finite.lean,Mathlib/Combinatorics/SimpleGraph/Copy.lean,Mathlib/Combinatorics/SimpleGraph/Regularity/Uniform.lean,Mathlib/Data/Finset/Card.lean,Mathlib/Data/Nat/Squarefree.lean,Mathlib/MeasureTheory/Integral/Bochner/VitaliCaratheodory.lean,Mathlib/RingTheory/Polynomial/Pochhammer.lean,Mathlib/Topology/ContinuousMap/Polynomial.lean |
14 |
9 |
['JovanGerb', 'eric-wieser', 'github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
12-1853 12 days ago |
12-1853 12 days ago |
0-0 0 seconds |
25969 |
101damnations author:101damnations |
feat(RepresentationTheory/Homological/GroupHomology/Functoriality): the degree 1 part of the corestriction-coinflation exact sequence |
Given a `G`-representation `A` and a normal subgroup `S` of `G`, this PR defines the corestriction-coinflation short complex
`H₁(S, A) ⟶ H₁(G, A) ⟶ H₁(G ⧸ S, A_S)` induced by the natural inclusion `S → G` and projections `G → G / S, A → A_S`. We prove it's exact, and that the righthand map is an epimorphism.
---
- [x] depends on: #21652
- [x] depends on: #21732
- [x] depends on: #21733
- [x] depends on: #21735
- [x] depends on: #21736
- [x] depends on: #21738
- [x] depends on: #25868
- [x] depends on: #25873
- [x] depends on: #25880
- [x] depends on: #25884
- [x] depends on: #25888
- [x] depends on: #25939
- [x] depends on: #25952
[](https://gitpod.io/from-referrer/)
---
*Earlier version at #22656.*
|
t-algebra
awaiting-author
label:t-algebra$ |
227/4 |
Mathlib/Algebra/Homology/ShortComplex/ModuleCat.lean,Mathlib/RepresentationTheory/Coinvariants.lean,Mathlib/RepresentationTheory/Homological/GroupHomology/Basic.lean,Mathlib/RepresentationTheory/Homological/GroupHomology/Functoriality.lean,Mathlib/RepresentationTheory/Homological/GroupHomology/LowDegree.lean |
5 |
n/a |
['github-actions', 'jcommelin', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
11-82994 11 days ago |
unknown |
unknown |
22231 |
pechersky author:pechersky |
feat(Algebra/Valued): `AdicExpansion` initial defns |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-topology
awaiting-author
label:t-algebra$ |
299/0 |
Mathlib.lean,Mathlib/Topology/Algebra/Valued/AdicExpansion.lean |
2 |
7 |
['Thmoas-Guan', 'github-actions', 'grunweg', 'jcommelin'] |
jcommelin assignee:jcommelin |
11-80625 11 days ago |
11-80625 11 days ago |
189-33553 189 days |
26101 |
xroblot author:xroblot |
feat(NumberField): specialized version of Kummer Dedekind for the splitting of prime numbers |
We prove a specialized version of [KummerDedekind.normalizedFactorsMapEquivNormalizedFactorsMinPolyMk](https://leanprover-community.github.io/mathlib4_docs/Mathlib/NumberTheory/KummerDedekind.html#KummerDedekind.normalizedFactorsMapEquivNormalizedFactorsMinPolyMk) for the splitting of rational prime numbers in number fields.
This PR continues the work from #25038.
---
- [x] depends on: #26137 |
t-number-theory |
172/1 |
Mathlib/NumberTheory/NumberField/Ideal/KummerDedekind.lean,Mathlib/NumberTheory/RamificationInertia/Basic.lean,Mathlib/RingTheory/AdjoinRoot.lean,Mathlib/RingTheory/DedekindDomain/Ideal/Lemmas.lean |
4 |
6 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'xroblot'] |
tb65536 assignee:tb65536 |
11-78621 11 days ago |
27-9959 27 days ago |
0-50 50 seconds |
29151 |
yuanyi-350 author:yuanyi-350 |
feat: Corollary of Hahn-Banach theorem |
In this PR, I have proved [Rudin, *Functional Analysis* (Theorem 3.7)][rudin1991] which is a step in proving the Closed Range Theorem. Also, I have added tags for the corresponding theorems in Rudin to mathlib.
3.7 Theorem. Suppose B is a convex, balanced, closed set in a locally convex space $X, x_0 \in X$, but $x_0 \notin B$. Then there exists $\Lambda \in X^*$ such that $|\Lambda x| \leq 1$ for all $x \in B$, but $\Lambda x_0>1$
proof. Since $B$ is closed and convex, we can apply (b) of Theorem 3.4, with $A=\{ x_0 \}$ , to obtain $\Lambda_1 \in X^*$ such that $\Lambda_1 x_0=r e^{i \theta}$ lies outside the closure $K$ of $\Lambda_1(B)$. Since $B$ is balanced, so is $K$. Hence there exists $s, 0" --allow-empty -m "add Author Name as coauthor"
When merging, all the commits will be squashed into a single commit listing all co-authors.
If you are moving or deleting declarations, please include these lines at the bottom of the commit message
(that is, before the `---`) using the following format:
Moves:
- Vector.* -> List.Vector.*
- ...
Deletions:
- Nat.bit1_add_bit1
- ...
Any other comments you want to keep out of the PR commit should go
below the `---`, and placed outside this HTML comment, or else they
will be invisible to reviewers.
If this PR depends on other PRs, please list them below this comment,
using the following format:
- [ ] depends on: #abc [optional extra text]
- [ ] depends on: #xyz [optional extra text]
-->
[](https://gitpod.io/from-referrer/)
|
large-import |
82/4 |
Mathlib/Analysis/NormedSpace/HahnBanach/Separation.lean,Mathlib/Topology/Order/OrderClosed.lean |
2 |
1 |
['github-actions'] |
faenuccio assignee:faenuccio |
11-77486 11 days ago |
13-22615 13 days ago |
13-38492 13 days |
27363 |
101damnations author:101damnations |
feat(RepresentationTheory/Homological): add standard resolution for finite cyclic groups |
Let `k` be a commutative ring and `G` a finite commutative group. Given `g : G` and `A : Rep k G`, we can define a periodic chain complex in `Rep k G` given by `... ⟶ A --N--> A --(ρ(g) - 𝟙)--> A --N--> A --(ρ(g) - 𝟙)--> A ⟶ 0` where `N` is the norm map sending `a : A` to `∑ ρ(g)(a)` for all `g` in `G`.
When `G` is generated by `g` and `A` is the left regular representation `k[G]`, this chain complex is a projective resolution of `k` as a trivial representation, which we prove in this PR.
---
- [x] depends on: #27362
- [x] depends on: #27361
[](https://gitpod.io/from-referrer/)
|
t-algebra
delegated
label:t-algebra$ |
223/0 |
Mathlib.lean,Mathlib/RepresentationTheory/Homological/FiniteCyclic.lean,Mathlib/RepresentationTheory/Invariants.lean |
3 |
10 |
['github-actions', 'jcommelin', 'mathlib-bors', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'sgouezel'] |
TwoFX assignee:TwoFX |
11-77277 11 days ago |
11-77277 11 days ago |
25-65075 25 days |
28452 |
plp127 author:plp127 |
feat: Define `ZMod.fintype` without cases |
Define `ZMod.fintype` without casing on `n` except inside the proof.
---
[](https://gitpod.io/from-referrer/)
|
t-data |
2/3 |
Mathlib/Data/ZMod/Defs.lean |
1 |
2 |
['github-actions', 'jcommelin'] |
nobody |
11-76441 11 days ago |
29-29960 29 days ago |
29-30003 29 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
delegated
|
30/19 |
Mathlib/Topology/Homotopy/Basic.lean,Mathlib/Topology/Homotopy/Contractible.lean,Mathlib/Topology/Homotopy/Equiv.lean,Mathlib/Topology/Homotopy/Lifting.lean |
4 |
7 |
['github-actions', 'grunweg', 'jcommelin', 'mathlib-bors', 'urkud'] |
grunweg assignee:grunweg |
11-75306 11 days ago |
11-75306 11 days ago |
111-33879 111 days |
28234 |
alreadydone author:alreadydone |
chore(AlgebraicTopology): clean up FundamentalGroupoid |
+ 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. This requires fixing some proofs about `HomotopyGroup`s, so we take this opportunity to golf a few proofs and replace `=>` by `↦`.
+ Golf within the file FundamentalGroupoid/Basic.
+ Generalize `toArrow` up to `fromPath` in `FundamentalGroupoid/FundamentalGroup` from `X : TopCat` to `[TopologicalSpace X]`.
---
[](https://gitpod.io/from-referrer/)
|
t-algebraic-topology
awaiting-author
|
104/141 |
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/Product.lean |
8 |
3 |
['github-actions', 'jcommelin', 'mathlib4-merge-conflict-bot'] |
mattrobball assignee:mattrobball |
11-73890 11 days ago |
11-73890 11 days ago |
20-65201 20 days |
28321 |
kim-em author:kim-em |
chore: make OmegaCompletePartialOrder a mixin |
I've noted typeclass searches often getting distracted looking for a `OmegaCompletePartialOrder` when they just want an `LE` or a `Preorder`.
Let's benchmark to see it if has a nontrivial effect. Not certain if this is desirable if the performance change is neutral (or even negative). |
awaiting-author |
68/43 |
Mathlib/Control/LawfulFix.lean,Mathlib/Data/Nat/Nth.lean,Mathlib/LinearAlgebra/AffineSpace/AffineSubspace/Defs.lean,Mathlib/Order/Category/OmegaCompletePartialOrder.lean,Mathlib/Order/OmegaCompletePartialOrder.lean,Mathlib/Topology/OmegaCompletePartialOrder.lean |
6 |
5 |
['github-actions', 'jcommelin', 'leanprover-bot', 'leanprover-community-mathlib4-bot'] |
nobody |
11-70034 11 days ago |
11-70034 11 days ago |
19-47454 19 days |
29147 |
ocfnash author:ocfnash |
feat: miscellaneous root system lemmas |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
WIP
label:t-algebra$ |
73/34 |
Mathlib/LinearAlgebra/RootSystem/Defs.lean,Mathlib/LinearAlgebra/RootSystem/Finite/G2.lean,Mathlib/LinearAlgebra/RootSystem/Finite/Nondegenerate.lean,Mathlib/LinearAlgebra/RootSystem/Reduced.lean |
4 |
1 |
['github-actions'] |
nobody |
11-65410 11 days ago |
13-50070 13 days ago |
0-2 2 seconds |
28702 |
Timeroot author:Timeroot |
feat(Algebra/Group/Hom/Defs): MonoidHom switching from MulOneClass to MulOne |
Currently `MonoidHom` relies on a `MulOneClass`, stating that 1 is a multiplicative identity; when actually all a "monoid" hom does is preserve multiplication and one. So, really, a MonoidHom is a "mul-and-one hom", but one cannot use it with any type that isn't a MulOneClass. (It also does not enforce being a Monoid: associativity is not required.)
In general, homs like this should only rely on the data being present in the source and destination type; any applications of it are then free to assume MulOneClass or Monoid where appropriate, which is essentially already how it does. This drops the MulOneClass assumption so that MonoidHom just takes the Mul and One types.
_But_ if we wrote `MonoidHom [Mul M] [One M]`, this would essentially double the effort needed for typeclass inference. An experiment in #28889 confirmed this performance hit. So, we define a `MulOne` type which is just the `Mul` and `One` data bundled together, and the performance change becomes pretty minimal.
And then there are the corresponding changes to `AddMonoidHom` / `AddZeroClass` becoming `AddZero`. This follows some discussion at [#mathlib4 > RingHom for not-a-ring](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/RingHom.20for.20not-a-ring)
---
[](https://gitpod.io/from-referrer/)
|
bench-after-CI
t-algebra
label:t-algebra$ |
78/68 |
Mathlib/Algebra/Group/Defs.lean,Mathlib/Algebra/Group/Ext.lean,Mathlib/Algebra/Group/Hom/Defs.lean,Mathlib/Algebra/Ring/Ext.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Affine/Point.lean,Mathlib/LinearAlgebra/LinearPMap.lean,Mathlib/RingTheory/Kaehler/JacobiZariski.lean |
7 |
5 |
['Timeroot', 'github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot'] |
dagurtomas assignee:dagurtomas |
11-63941 11 days ago |
20-26134 20 days ago |
23-60330 23 days |
26710 |
metakunt author:metakunt |
feat (Data/Nat/Digits/Lemmas): Add digits_getD |
Adds digits_getD, an explicit computation of the i-th digits of n in base b representation. |
t-data
new-contributor
awaiting-author
|
48/0 |
Mathlib/Data/Nat/Digits/Lemmas.lean |
1 |
8 |
['github-actions', 'pechersky', 'plp127'] |
nobody |
11-53113 11 days ago |
14-52304 14 days ago |
56-72456 56 days |
28070 |
grunweg author:grunweg |
style: improve indentation of multi-linear enumerations in doc-strings |
Per zulip discussion: [#mathlib4 > Style :bicycle: : indenting second lines in doc-strings @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Style.20.3Abicycle.3A.20.3A.20indenting.20second.20lines.20in.20doc-strings/near/533105734).
---
[](https://gitpod.io/from-referrer/)
|
|
111/108 |
Archive/Wiedijk100Theorems/SumOfPrimeReciprocalsDiverges.lean,Mathlib/Algebra/Algebra/Defs.lean,Mathlib/Algebra/BrauerGroup/Defs.lean,Mathlib/Algebra/Module/LinearMap/Polynomial.lean,Mathlib/CategoryTheory/Abelian/NonPreadditive.lean,Mathlib/CategoryTheory/EqToHom.lean,Mathlib/CategoryTheory/Filtered/Basic.lean,Mathlib/CategoryTheory/Limits/Final.lean,Mathlib/CategoryTheory/Limits/Pi.lean,Mathlib/CategoryTheory/Monoidal/Center.lean,Mathlib/CategoryTheory/Sites/Grothendieck.lean,Mathlib/CategoryTheory/Sites/Pretopology.lean,Mathlib/Condensed/Discrete/Characterization.lean,Mathlib/FieldTheory/ChevalleyWarning.lean,Mathlib/GroupTheory/MonoidLocalization/Basic.lean,docs/Conv/Guide.lean |
16 |
6 |
['github-actions', 'grunweg', 'kbuzzard'] |
kbuzzard assignee:kbuzzard |
11-51053 11 days ago |
37-11189 1 month ago |
37-11169 37 days |
27973 |
smmercuri author:smmercuri |
feat: the ring of integers of a `ℤₘ₀`-valued field is compact whenever it is a DVR and the residue field is finite |
This PR continues the work from #21844.
Original PR: https://github.com/leanprover-community/mathlib4/pull/21844 |
large-import
t-algebra
label:t-algebra$ |
54/2 |
Mathlib/RingTheory/Ideal/Quotient/Basic.lean,Mathlib/Topology/Algebra/Valued/WithZeroMulInt.lean |
2 |
1 |
['github-actions'] |
dagurtomas assignee:dagurtomas |
11-34918 11 days ago |
21-19967 21 days ago |
31-65206 31 days |
28602 |
gmcninch-tufts author:gmcninch-tufts |
feat(Algebra/Polynomial/Module): prove equivalence of a certain tensor product with PolynomialModule |
For a commutative ring `R` and an `R`-module `M`, construct an equivalence between the `R[X]`-modules `R[X] ⊗[R] M` and
`PolynomialModule R M`.
This equivalence enables application of some base-change results to `PolynomialModule R M` .
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-algebra
label:t-algebra$ |
210/0 |
Mathlib.lean,Mathlib/Algebra/Polynomial/Module/TensorProduct.lean |
2 |
1 |
['github-actions'] |
jcommelin assignee:jcommelin |
11-34916 11 days ago |
25-70392 25 days ago |
25-70433 25 days |
23992 |
robertmaxton42 author:robertmaxton42 |
feat (Limits.FunctorCategory): limitIsoFlipCompLim and colimitIsoFlipCompColim are natural |
Add `limIsoFlipCompWhiskerLim`, `limCompFlipIsoWhiskerLim`, `colimIsoFlipCompWhiskerColim`, `colimCompFlipIsoWhiskerColim`, each witnessing that their corresponding families of isomorphisms are natural in the diagram $F$.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-category-theory
awaiting-CI
|
41/0 |
Mathlib/CategoryTheory/Limits/FunctorCategory/Basic.lean |
1 |
13 |
['adomani', 'github-actions', 'robertmaxton42', 'robin-carlier'] |
nobody |
11-34578 11 days ago |
99-42180 3 months ago |
50-83251 50 days |
28934 |
yury-harmonic author:yury-harmonic |
feat(NormNum): add extensions for `Even` and `Odd` |
---
[](https://gitpod.io/from-referrer/)
|
maintainer-merge
t-meta
awaiting-author
|
55/0 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/NormNum/Parity.lean,scripts/noshake.json |
4 |
10 |
['JovanGerb', 'adomani', 'digama0', 'github-actions', 'mathlib4-merge-conflict-bot', 'yury-harmonic'] |
nobody |
11-33439 11 days ago |
11-50507 11 days ago |
6-16639 6 days |
29231 |
kim-em author:kim-em |
chore: deprecate PartENat |
See [#mathlib4 > deprecate Mathlib.Data.Nat.PartENat?](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/deprecate.20Mathlib.2EData.2ENat.2EPartENat.3F). |
t-data |
7/0 |
Mathlib/Data/Nat/PartENat.lean |
1 |
1 |
['github-actions'] |
nobody |
11-27446 11 days ago |
11-27664 11 days ago |
11-27710 11 days |
19860 |
YaelDillies author:YaelDillies |
refactor: review the `simps` projections of `OneHom`, `MulHom`, `MonoidHom` |
Make `simps` generate `coe_concreteHom` rather than`concreteHom_apply`.
From FLT
---
In fact, I would love to have both the `coe_` and `_apply` projections simultaneously and also to not have to specify ` simps (config := .asFn))` every single time we want to generate the `coe_` projection, but `simps ` seems to not be able to do that? cc @fpvandoorn
I must say, after four years of working on mathlib, I still don't understand how one is supposed to use `simps`.
[](https://gitpod.io/from-referrer/)
|
t-algebra
WIP
label:t-algebra$ |
104/119 |
Mathlib/Algebra/BigOperators/Group/Multiset/Basic.lean,Mathlib/Algebra/Group/Hom/Defs.lean,Mathlib/Algebra/Group/Subgroup/Defs.lean,Mathlib/Algebra/Group/Submonoid/Operations.lean,Mathlib/Algebra/Group/WithOne/Basic.lean,Mathlib/Algebra/GroupWithZero/WithZero.lean,Mathlib/Algebra/Module/End.lean,Mathlib/GroupTheory/NoncommCoprod.lean |
8 |
10 |
['fpvandoorn', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-merge-conflict-bot'] |
nobody |
10-72419 10 days ago |
10-72444 10 days ago |
0-17 17 seconds |
27500 |
Komyyy author:Komyyy |
feat: the Riemann zeta function is meromorphic |
Also proves that the Hurwitz zeta function is meromorphic. This PR is split from #27499 to leave a good git diff history.
---
The `large-import` change occurs only in the new module, so it poses no problem.
- [x] depends on: #27499
This PR continues the work from #25597.
Original PR: https://github.com/leanprover-community/mathlib4/pull/25597 |
large-import
t-analysis
WIP
|
51/3 |
Mathlib.lean,Mathlib/Analysis/Meromorphic/Complex.lean,Mathlib/Analysis/Meromorphic/Gamma.lean |
3 |
13 |
['Komyyy', 'github-actions', 'j-loreaux', 'loefflerd', 'mathlib4-dependent-issues-bot'] |
j-loreaux assignee:j-loreaux |
10-65066 10 days ago |
15-71914 15 days ago |
30-62878 30 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 |
5 |
['b-mehta', 'github-actions', 'grunweg', 'plp127'] |
b-mehta assignee:b-mehta |
10-63646 10 days ago |
82-22088 2 months ago |
82-36000 82 days |
25814 |
vlad902 author:vlad902 |
feat(SimpleGraph): Weaker condition for paths in acyclic graphs |
`IsAcyclic.isPath_iff_chain'` defines a weaker condition for proving that a walk is a path, in particular it shows that rather than proving that all vertices in the support of a walk are distinct, one must only show that consecutive edges are distinct (e.g. every other vertex must be distinct.) This leads to a simple corollary that trails are also paths in acyclic graphs.
I had a need for this when formalizing Cayley graphs, since this condition maps cleanly onto words in free groups being reduced.
---
*This PR continues the work from #25630.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/25630* |
t-combinatorics |
42/0 |
Mathlib/Combinatorics/SimpleGraph/Acyclic.lean,Mathlib/Combinatorics/SimpleGraph/Paths.lean |
2 |
2 |
['github-actions', 'vlad902'] |
kmill assignee:kmill |
10-63567 10 days ago |
92-73503 3 months ago |
92-73483 92 days |
29207 |
YaelDillies author:YaelDillies |
chore(MonoidAlgebra/Defs): reorder, rename variables |
Sort the declarations according to typeclass assumptions, *and* according to the order in which we need them to be for #25273.
Rename the semiring variable to `R` and the monoid one to `M`.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
awaiting-CI
help-wanted
label:t-algebra$ |
458/586 |
Mathlib/Algebra/MonoidAlgebra/Basic.lean,Mathlib/Algebra/MonoidAlgebra/Defs.lean,Mathlib/Algebra/MonoidAlgebra/Division.lean,Mathlib/Algebra/MonoidAlgebra/Grading.lean,Mathlib/Algebra/MonoidAlgebra/Module.lean,Mathlib/Algebra/MvPolynomial/Basic.lean,Mathlib/Algebra/Polynomial/Laurent.lean |
7 |
2 |
['YaelDillies', 'github-actions'] |
nobody |
10-63210 10 days ago |
10-63210 10 days ago |
0-7 7 seconds |
23940 |
YaelDillies author:YaelDillies |
feat: polytopes |
From Toric
Co-authored-by: Matthew Johnson
---
[](https://gitpod.io/from-referrer/)
|
toric
t-analysis
awaiting-author
|
65/0 |
Mathlib.lean,Mathlib/Geometry/Convex/Polytope.lean,Mathlib/Geometry/Convex/README.md |
3 |
11 |
['Parcly-Taxel', 'YaelDillies', 'eric-wieser', 'github-actions', 'j-loreaux', 'jsm28', 'leanprover-community-bot-assistant', 'ooovi'] |
j-loreaux assignee:j-loreaux |
10-62715 10 days ago |
10-62731 10 days ago |
143-64212 143 days |
26051 |
Komyyy author:Komyyy |
feat(Mathlib/GroupTheory/SpecificGroups/Alternating): A_n is simple iff n = 3 or 5 ≤ n |
---
- [x] depends on: #25299
- [x] depends on: #25314
- [x] depends on: #25367
- [x] depends on: #26098
- [x] depends on: #26552
- [x] depends on: #27498
- [x] depends on: #29234
This PR continues the work from #23555.
Original PR: https://github.com/leanprover-community/mathlib4/pull/23555
[](https://gitpod.io/from-referrer/) |
t-group-theory
large-import
WIP
|
290/71 |
Mathlib.lean,Mathlib/GroupTheory/SpecificGroups/Alternating.lean,Mathlib/GroupTheory/SpecificGroups/Alternating/Simple.lean,Mathlib/GroupTheory/Subgroup/Simple.lean |
4 |
13 |
['Komyyy', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'tb65536'] |
nobody |
10-58965 10 days ago |
10-75623 10 days ago |
10-66608 10 days |
25780 |
emilyriehl author:emilyriehl |
feat: the homotopy category functor preserves products |
This proves that the homotopy category construction defines a lax monoidal functor from simplicial sets to categories. In particular, simplicially enriched categories have quotient categorically enriched categories, which might be thought of as "homotopy bicategories."
Co-authored-by: Dominic Verity , Bhavik Mehta , Thomas Murrills , and Andrew Yang .
---
- [x] depends on: #27576
*This PR continues the work from #25010.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/25010* |
t-algebraic-topology
infinity-cosmos
large-import
t-category-theory
|
253/11 |
Mathlib/AlgebraicTopology/SimplexCategory/Defs.lean,Mathlib/AlgebraicTopology/SimplicialSet/Nerve.lean,Mathlib/AlgebraicTopology/SimplicialSet/NerveAdjunction.lean,Mathlib/AlgebraicTopology/SimplicialSet/StdSimplex.lean,Mathlib/CategoryTheory/Category/ULift.lean,Mathlib/CategoryTheory/ComposableArrows.lean,Mathlib/CategoryTheory/Limits/Preserves/Basic.lean,Mathlib/CategoryTheory/Limits/Shapes/BinaryProducts.lean,Mathlib/CategoryTheory/Monoidal/Cartesian/Basic.lean,Mathlib/Order/Hom/Basic.lean |
10 |
6 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
10-45973 10 days ago |
25-75286 25 days ago |
25-76331 25 days |
28429 |
euprunin author:euprunin |
chore(GroupTheory/Perm/Cycle): deprecate `Disjoint.cycleType_mul` |
---
[](https://gitpod.io/from-referrer/)
|
t-group-theory
awaiting-author
|
2/8 |
Mathlib/GroupTheory/Perm/Cycle/Type.lean |
1 |
4 |
['euprunin', 'github-actions', 'tb65536'] |
tb65536 assignee:tb65536 |
10-45142 10 days ago |
15-59976 15 days ago |
12-12845 12 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 |
2 |
['artie2000', 'github-actions'] |
joneugster assignee:joneugster |
10-35422 10 days ago |
81-69365 2 months ago |
85-40611 85 days |
27238 |
alreadydone author:alreadydone |
feat(Algebra): IsDomain R[X] ↔ IsDomain R ∧ IsCancelAdd R |
---
- [x] depends on: #27241
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
133/1 |
Counterexamples.lean,Counterexamples/PolynomialIsDomain.lean,Mathlib/Algebra/Group/Defs.lean,Mathlib/Algebra/Group/Opposite.lean,Mathlib/Algebra/GroupWithZero/TransferInstance.lean,Mathlib/Algebra/Opposites.lean,Mathlib/Algebra/Polynomial/Basic.lean,Mathlib/RingTheory/Polynomial/Opposites.lean |
8 |
7 |
['alreadydone', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
kim-em assignee:kim-em |
10-34926 10 days ago |
21-39150 21 days ago |
25-24940 25 days |
28564 |
euprunin author:euprunin |
chore(LinearAlgebra): golf entire `congr_symm`, `LinearMap.toMatrix_smulBasis_left`, `LinearMap.toMatrix_smulBasis_right` and more using `rfl` |
---
Show trace profiling of congr_symm : 24 ms before, 28 ms after
### Trace profiling of `congr_symm` before PR 28564
```diff
diff --git a/Mathlib/LinearAlgebra/BilinearForm/Hom.lean b/Mathlib/LinearAlgebra/BilinearForm/Hom.lean
index c056a51a5b..90cb2cd345 100644
--- a/Mathlib/LinearAlgebra/BilinearForm/Hom.lean
+++ b/Mathlib/LinearAlgebra/BilinearForm/Hom.lean
@@ -204,6 +204,7 @@ theorem congr_apply (e : M ≃ₗ[R] M') (B : BilinForm R M) (x y : M') :
congr e B x y = B (e.symm x) (e.symm y) :=
rfl
+set_option trace.profiler true in
@[simp]
theorem congr_symm (e : M ≃ₗ[R] M') : (congr e).symm = congr e.symm := by
ext
```
```
ℹ [1062/1062] Built Mathlib.LinearAlgebra.BilinearForm.Hom (3.4s)
info: Mathlib/LinearAlgebra/BilinearForm/Hom.lean:208:0: [Elab.command] [0.026792] @[simp]
theorem congr_symm (e : M ≃ₗ[R] M') : (congr e).symm = congr e.symm :=
by
ext
simp only [congr_apply, LinearEquiv.symm_symm]
rfl
info: Mathlib/LinearAlgebra/BilinearForm/Hom.lean:208:0: [Elab.async] [0.024764] elaborating proof of LinearMap.BilinForm.congr_symm
[Elab.definition.value] [0.023696] LinearMap.BilinForm.congr_symm
[Elab.step] [0.022888]
ext
simp only [congr_apply, LinearEquiv.symm_symm]
rfl
[Elab.step] [0.022873]
ext
simp only [congr_apply, LinearEquiv.symm_symm]
rfl
info: Mathlib/LinearAlgebra/BilinearForm/Hom.lean:209:8: [Elab.async] [0.011246] Lean.addDecl
[Kernel] [0.011207] ✅️ typechecking declarations [LinearMap.BilinForm.congr_symm]
Build completed successfully (1062 jobs).
```
### Trace profiling of `congr_symm` after PR 28564
```diff
diff --git a/Mathlib/LinearAlgebra/BilinearForm/Hom.lean b/Mathlib/LinearAlgebra/BilinearForm/Hom.lean
index c056a51a5b..ce976f69d7 100644
--- a/Mathlib/LinearAlgebra/BilinearForm/Hom.lean
+++ b/Mathlib/LinearAlgebra/BilinearForm/Hom.lean
@@ -204,11 +204,10 @@ theorem congr_apply (e : M ≃ₗ[R] M') (B : BilinForm R M) (x y : M') :
congr e B x y = B (e.symm x) (e.symm y) :=
rfl
+set_option trace.profiler true in
@[simp]
theorem congr_symm (e : M ≃ₗ[R] M') : (congr e).symm = congr e.symm := by
- ext
- simp only [congr_apply, LinearEquiv.symm_symm]
- rfl
+ tauto
@[simp]
theorem congr_refl : congr (LinearEquiv.refl R M) = LinearEquiv.refl R _ :=
diff --git a/Mathlib/LinearAlgebra/Matrix/ToLin.lean b/Mathlib/LinearAlgebra/Matrix/ToLin.lean
index e78673e1fa..b05d64e287 100644
--- a/Mathlib/LinearAlgebra/Matrix/ToLin.lean
+++ b/Mathlib/LinearAlgebra/Matrix/ToLin.lean
@@ -681,17 +681,13 @@ theorem LinearMap.toMatrix_smulBasis_left {G} [Group G] [DistribMulAction G M₁
[SMulCommClass G R M₁] (g : G) (f : M₁ →ₗ[R] M₂) :
LinearMap.toMatrix (g • v₁) v₂ f =
LinearMap.toMatrix v₁ v₂ (f ∘ₗ DistribMulAction.toLinearMap _ _ g) := by
- ext
- rw [LinearMap.toMatrix_apply, LinearMap.toMatrix_apply]
- dsimp
+ tauto
theorem LinearMap.toMatrix_smulBasis_right {G} [Group G] [DistribMulAction G M₂]
[SMulCommClass G R M₂] (g : G) (f : M₁ →ₗ[R] M₂) :
LinearMap.toMatrix v₁ (g • v₂) f =
LinearMap.toMatrix v₁ v₂ (DistribMulAction.toLinearMap _ _ g⁻¹ ∘ₗ f) := by
- ext
- rw [LinearMap.toMatrix_apply, LinearMap.toMatrix_apply]
- dsimp
+ tauto
end Finite
diff --git a/Mathlib/LinearAlgebra/Multilinear/Curry.lean b/Mathlib/LinearAlgebra/Multilinear/Curry.lean
index dbccfc807a..9175992b1f 100644
--- a/Mathlib/LinearAlgebra/Multilinear/Curry.lean
+++ b/Mathlib/LinearAlgebra/Multilinear/Curry.lean
@@ -84,9 +84,7 @@ theorem MultilinearMap.curryLeft_apply (f : MultilinearMap R M M₂) (x : M 0)
@[simp]
theorem LinearMap.curry_uncurryLeft (f : M 0 →ₗ[R] MultilinearMap R (fun i :
Fin n => M i.succ) M₂) : f.uncurryLeft.curryLeft = f := by
- ext m x
- simp only [tail_cons, LinearMap.uncurryLeft_apply, MultilinearMap.curryLeft_apply]
- rw [cons_zero]
+ tauto
@[simp]
theorem MultilinearMap.uncurry_curryLeft (f : MultilinearMap R M M₂) :
diff --git a/Mathlib/LinearAlgebra/TensorProduct/Graded/External.lean b/Mathlib/LinearAlgebra/TensorProduct/Graded/External.lean
index 140f4599b3..a5fc97375b 100644
--- a/Mathlib/LinearAlgebra/TensorProduct/Graded/External.lean
+++ b/Mathlib/LinearAlgebra/TensorProduct/Graded/External.lean
@@ -104,9 +104,7 @@ def gradedComm :
/-- The braiding is symmetric. -/
@[simp]
theorem gradedComm_symm : (gradedComm R 𝒜 ℬ).symm = gradedComm R ℬ 𝒜 := by
- rw [gradedComm, gradedComm, LinearEquiv.trans_symm, LinearEquiv.symm_symm]
- ext
- rfl
+ tauto
theorem gradedComm_of_tmul_of (i j : ι) (a : 𝒜 i) (b : ℬ j) :
gradedComm R 𝒜 ℬ (lof R _ 𝒜 i a ⊗ₜ lof R _ ℬ j b) =
```
```
ℹ [1062/1062] Built Mathlib.LinearAlgebra.BilinearForm.Hom (3.4s)
info: Mathlib/LinearAlgebra/BilinearForm/Hom.lean:208:0: [Elab.command] [0.022737] @[simp]
theorem congr_symm (e : M ≃ₗ[R] M') : (congr e).symm = congr e.symm := by tauto
info: Mathlib/LinearAlgebra/BilinearForm/Hom.lean:208:0: [Elab.async] [0.030155] elaborating proof of LinearMap.BilinForm.congr_symm
[Elab.definition.value] [0.028158] LinearMap.BilinForm.congr_symm
[Elab.step] [0.027405] tauto
[Elab.step] [0.027386] tauto
[Elab.step] [0.027369] tauto
[Elab.step] [0.019442] rfl
[Elab.step] [0.019158] eq_refl
[Meta.isDefEq] [0.019142] ✅️ (congr e).symm =?= congr e.symm
[Meta.isDefEq] [0.019026] ✅️ (congr
e).symm =?= (LinearEquiv.congrLeft R R e.symm).congrRight.trans
(LinearEquiv.congrLeft (M →ₗ[R] R) R e.symm)
[Meta.isDefEq] [0.018960] ✅️ have __src := (↑(congr e)).inverse (congr e).invFun ⋯ ⋯;
let __src := (congr e).toEquiv.symm;
{ toFun := ⇑((↑(congr e)).inverse (congr e).invFun ⋯ ⋯), map_add' := ⋯, map_smul' := ⋯,
invFun := (congr e).toEquiv.symm.invFun, left_inv := ⋯,
right_inv :=
⋯ } =?= (LinearEquiv.congrLeft R R e.symm).congrRight.trans
(LinearEquiv.congrLeft (M →ₗ[R] R) R e.symm)
[Meta.isDefEq] [0.018936] ✅️ { toFun := ⇑((↑(congr e)).inverse (congr e).invFun ⋯ ⋯), map_add' := ⋯,
map_smul' := ⋯, invFun := (congr e).toEquiv.symm.invFun, left_inv := ⋯,
right_inv :=
⋯ } =?= (LinearEquiv.congrLeft R R e.symm).congrRight.trans
(LinearEquiv.congrLeft (M →ₗ[R] R) R e.symm)
[Meta.isDefEq] [0.018834] ✅️ { toFun := ⇑((↑(congr e)).inverse (congr e).invFun ⋯ ⋯),
map_add' := ⋯, map_smul' := ⋯, invFun := (congr e).toEquiv.symm.invFun, left_inv := ⋯,
right_inv :=
⋯ } =?= let __src :=
↑(LinearEquiv.congrLeft (M →ₗ[R] R) R e.symm) ∘ₗ
↑(LinearEquiv.congrLeft R R e.symm).congrRight;
let __src_1 :=
(LinearEquiv.congrLeft R R e.symm).congrRight.toEquiv.trans
(LinearEquiv.congrLeft (M →ₗ[R] R) R e.symm).toEquiv;
{ toLinearMap := __src, invFun := __src_1.invFun, left_inv := ⋯, right_inv := ⋯ }
[Meta.isDefEq] [0.018825] ✅️ { toFun := ⇑((↑(congr e)).inverse (congr e).invFun ⋯ ⋯),
map_add' := ⋯, map_smul' := ⋯, invFun := (congr e).toEquiv.symm.invFun, left_inv := ⋯,
right_inv :=
⋯ } =?= {
toLinearMap :=
↑(LinearEquiv.congrLeft (M →ₗ[R] R) R e.symm) ∘ₗ
↑(LinearEquiv.congrLeft R R e.symm).congrRight,
invFun :=
((LinearEquiv.congrLeft R R e.symm).congrRight.toEquiv.trans
(LinearEquiv.congrLeft (M →ₗ[R] R) R e.symm).toEquiv).invFun,
left_inv := ⋯, right_inv := ⋯ }
[Meta.isDefEq] [0.011340] ✅️ { toFun := ⇑((↑(congr e)).inverse (congr e).invFun ⋯ ⋯),
map_add' := ⋯,
map_smul' :=
⋯ } =?= ↑(LinearEquiv.congrLeft (M →ₗ[R] R) R e.symm) ∘ₗ
↑(LinearEquiv.congrLeft R R e.symm).congrRight
[Meta.isDefEq] [0.011274] ✅️ { toFun := ⇑((↑(congr e)).inverse (congr e).invFun ⋯ ⋯),
map_add' := ⋯,
map_smul' :=
⋯ } =?= {
toFun :=
⇑↑(LinearEquiv.congrLeft (M →ₗ[R] R) R e.symm) ∘
⇑↑(LinearEquiv.congrLeft R R e.symm).congrRight,
map_add' := ⋯, map_smul' := ⋯ }
[Meta.isDefEq] [0.010754] ✅️ { toFun := ⇑((↑(congr e)).inverse (congr e).invFun ⋯ ⋯),
map_add' :=
⋯ } =?= {
toFun :=
⇑↑(LinearEquiv.congrLeft (M →ₗ[R] R) R e.symm) ∘
⇑↑(LinearEquiv.congrLeft R R e.symm).congrRight,
map_add' := ⋯ }
info: Mathlib/LinearAlgebra/BilinearForm/Hom.lean:209:8: [Elab.async] [0.100749] Lean.addDecl
[Kernel] [0.100672] ✅️ typechecking declarations [LinearMap.BilinForm.congr_symm]
Build completed successfully (1062 jobs).
```
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
3/11 |
Mathlib/LinearAlgebra/BilinearForm/Hom.lean,Mathlib/LinearAlgebra/Matrix/ToLin.lean,Mathlib/LinearAlgebra/Multilinear/Curry.lean,Mathlib/LinearAlgebra/TensorProduct/Graded/External.lean |
4 |
4 |
['github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot'] |
joneugster assignee:joneugster |
10-34923 10 days ago |
17-40794 17 days ago |
25-80454 25 days |
28887 |
alreadydone author:alreadydone |
feat(RingTheory): units are exactly non-zerodivisors in noncommutative Artinian rings |
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
t-algebra
label:t-algebra$ |
70/24 |
Mathlib/RingTheory/Artinian/Algebra.lean,Mathlib/RingTheory/Artinian/Module.lean,Mathlib/RingTheory/Artinian/Ring.lean,Mathlib/RingTheory/IntegralClosure/IsIntegral/Basic.lean |
4 |
2 |
['github-actions', 'themathqueen'] |
mattrobball assignee:mattrobball |
10-34919 10 days ago |
17-48500 17 days ago |
19-32291 19 days |
28929 |
grunweg author:grunweg |
experiment: use `fun_prop` in Homeomorph |
Can we make the continuity auto-parameters use `fun_prop`?
Or perhaps `first |fun_prop; |dsimp; fun_prop`?
---
Compared to #13994, it seems this is a much smoother experience. I suspect the RefineDiscTree changes have helped (but that is pure speculation).
[](https://gitpod.io/from-referrer/)
|
t-topology |
13/5 |
Mathlib/MeasureTheory/Group/Measure.lean,Mathlib/Topology/Algebra/Algebra/Equiv.lean,Mathlib/Topology/Algebra/Constructions/DomMulAct.lean,Mathlib/Topology/Algebra/ContinuousMonoidHom.lean,Mathlib/Topology/Constructions/SumProd.lean,Mathlib/Topology/Homeomorph/Defs.lean |
6 |
4 |
['euprunin', 'github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot'] |
PatrickMassot assignee:PatrickMassot |
10-34919 10 days ago |
18-39197 18 days ago |
18-44514 18 days |
28973 |
YaelDillies author:YaelDillies |
feat(TensorProduct): `lTensor` as an `AlgHom` and other lemmas |
From Toric
Co-authored-by: Michał Mrugała
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
toric
|
21/0 |
Mathlib/RingTheory/TensorProduct/Basic.lean |
1 |
3 |
['github-actions', 'themathqueen'] |
mattrobball assignee:mattrobball |
10-34915 10 days ago |
17-68472 17 days ago |
17-68533 17 days |
29281 |
plp127 author:plp127 |
docs: `Fin.natAdd_castLEEmb` |
Change the docstring of `Fin.natAdd_castLEEmb` which confused me when I read it so I rewrote it.
PS. this doesn't really follow the naming convention since data should be in `camelCase`
---
[](https://gitpod.io/from-referrer/)
|
t-data |
2/3 |
Mathlib/Data/Fin/Embedding.lean |
1 |
1 |
['github-actions'] |
nobody |
10-30956 10 days ago |
10-30962 10 days ago |
10-31002 10 days |
29162 |
vlad902 author:vlad902 |
feat(SetTheory): generalize Schroeder-Bernstein theorem |
In a proof of the infinite-version of the graph theoretic statement of Hall's Marriage Theorem, I needed a slight generalization of the Schroeder-Bernstein theorem. In particular, I wanted the bijection to also satisfy a pointwise property that the individual injections satisfy. |
t-set-theory |
23/5 |
Mathlib/SetTheory/Cardinal/SchroederBernstein.lean |
1 |
11 |
['adomani', 'github-actions', 'grunweg', 'vihdzp', 'vlad902'] |
b-mehta assignee:b-mehta |
10-14786 10 days ago |
13-2107 13 days ago |
13-2147 13 days |
27308 |
xyzw12345 author:xyzw12345 |
feat(LinearAlgebra/SymmetricAlgebra): IsSymmetricAlgebra |
This PR continues the work from #24602.
Original PR: https://github.com/leanprover-community/mathlib4/pull/24602 |
t-algebra label:t-algebra$ |
78/0 |
Mathlib/LinearAlgebra/SymmetricAlgebra/Basic.lean,Mathlib/LinearAlgebra/SymmetricAlgebra/Basis.lean |
2 |
3 |
['github-actions', 'mattrobball', 'xyzw12345'] |
mattrobball assignee:mattrobball |
10-9025 10 days ago |
54-72249 1 month ago |
54-72298 54 days |
25927 |
jjdishere author:jjdishere |
feat(RingTheory/AdicCompletion): more APIs for IsAdicComplete |
This PR continues the work from #21582.
Original PR: https://github.com/leanprover-community/mathlib4/pull/21582 |
t-ring-theory
awaiting-author
|
452/11 |
Mathlib/RingTheory/AdicCompletion/Basic.lean,Mathlib/RingTheory/Ideal/Quotient/Defs.lean,Mathlib/RingTheory/Ideal/Quotient/PowTransition.lean |
3 |
5 |
['github-actions', 'jjdishere'] |
nobody |
10-8193 10 days ago |
39-3817 1 month ago |
9-35950 9 days |
27977 |
smmercuri author:smmercuri |
feat: predicates for extensions of complex embeddings |
This PR continues the work from #24877.
Original PR: https://github.com/leanprover-community/mathlib4/pull/24877 |
t-number-theory
WIP
|
91/0 |
Mathlib/NumberTheory/NumberField/InfinitePlace/Embeddings.lean |
1 |
4 |
['github-actions', 'riccardobrasca', 'smmercuri'] |
riccardobrasca assignee:riccardobrasca |
9-84208 9 days ago |
38-85664 1 month ago |
0-30 30 seconds |
29309 |
LLaurance author:LLaurance |
feat(Combinatorics/SimpleGraph): Nontrivial connected graph contains a vertex that leaves the graph connected if removed |
This shows that any nontrivial connected graph contains a vertex that, when removed, leaves the graph connected.
[](https://gitpod.io/from-referrer/)
|
large-import
new-contributor
t-combinatorics
|
156/10 |
Mathlib/Combinatorics/SimpleGraph/Acyclic.lean,Mathlib/Combinatorics/SimpleGraph/Connectivity/Connected.lean,Mathlib/Combinatorics/SimpleGraph/Connectivity/Subgraph.lean,Mathlib/Combinatorics/SimpleGraph/Subgraph.lean,Mathlib/Combinatorics/SimpleGraph/Walk.lean |
5 |
1 |
['github-actions'] |
nobody |
9-74074 9 days ago |
9-83827 9 days ago |
0-0 0 seconds |
29200 |
euprunin author:euprunin |
chore: remove redundant `simp_rw` invocations |
---
**Note:** Although technically redundant, some of these may be worth keeping for readability, or other reasons. Let me know if you think any should stay.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
awaiting-author
label:t-algebra$ |
0/12 |
Mathlib/Algebra/Algebra/Operations.lean,Mathlib/Algebra/Category/ModuleCat/Monoidal/Symmetric.lean,Mathlib/Algebra/Group/Pointwise/Set/BigOperators.lean,Mathlib/Algebra/Lie/Submodule.lean,Mathlib/Algebra/Lie/Weights/Chain.lean,Mathlib/Algebra/MvPolynomial/Degrees.lean,Mathlib/Algebra/Order/Antidiag/Pi.lean,Mathlib/Algebra/Order/BigOperators/Group/Multiset.lean |
8 |
16 |
['bryangingechen', 'euprunin', 'github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot'] |
nobody |
9-74049 9 days ago |
10-31679 10 days ago |
1-71534 1 day |
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
|
127/129 |
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/Enriched/Ordinary/Basic.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/Cartesian/Mon_.lean,Mathlib/CategoryTheory/Monoidal/Category.lean,Mathlib/CategoryTheory/Monoidal/DayConvolution.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/Basic.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 |
27 |
16 |
['YaelDillies', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-merge-conflict-bot', 'robin-carlier', 'yuma-mizuno'] |
kim-em assignee:kim-em |
9-73780 9 days ago |
10-72647 10 days ago |
74-40684 74 days |
29232 |
vihdzp author:vihdzp |
feat: more theorems on `SuccAddOrder` |
We make use of the (relatively) new `CanonicallyOrderedAdd` typeclass in order to generalize various theorems on `Ordinal` to `SuccAddOrder`. Later on we'll deprecate the `Ordinal` versions in favor of these.
---
[](https://gitpod.io/from-referrer/)
|
t-order
t-algebra
label:t-algebra$ |
54/1 |
Mathlib/Algebra/Order/SuccPred.lean |
1 |
2 |
['github-actions', 'plp127'] |
nobody |
9-67303 9 days ago |
11-24773 11 days ago |
11-24811 11 days |
27244 |
xroblot author:xroblot |
feat(RingTheory/DedekindDomain): lifting an ideal in an extension is injective |
This PR develops some API for [FractionalIdeal.extendedHomₐ](https://leanprover-community.github.io/mathlib4_docs/Mathlib/RingTheory/FractionalIdeal/Extended.html#FractionalIdeal.extendedHom%E2%82%90) and in particular proves when it is an injective map. As a consequence, it deduces the fact that lifting an integral ideal in an extension of Dedekind domains is an injective map.
Note: the import increase happens in a leaf file `Mathlib.RingTheory.FractionalIdeal.Extended`
---
- [x] depends on: #28800
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
large-import
|
140/8 |
Mathlib/RingTheory/DedekindDomain/Ideal/Lemmas.lean,Mathlib/RingTheory/FractionalIdeal/Extended.lean,Mathlib/RingTheory/Localization/Basic.lean |
3 |
5 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'xroblot'] |
kbuzzard assignee:kbuzzard |
9-66207 9 days ago |
9-77826 9 days ago |
45-82412 45 days |
27288 |
themathqueen author:themathqueen |
chore(LinearAlgebra/TensorProduct/Basic): semi-linearize `map` and `lift` |
Semi-linearizing `TensorProduct.map`.
Co-authored-by: Anatole Dedecker
---
Part of #27353.
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
40/27 |
Mathlib/Algebra/Category/ModuleCat/ChangeOfRings.lean,Mathlib/LinearAlgebra/TensorProduct/Basic.lean,Mathlib/RingTheory/Coalgebra/Hom.lean |
3 |
5 |
['ADedecker', 'eric-wieser', 'github-actions', 'themathqueen'] |
ADedecker assignee:ADedecker |
9-63743 9 days ago |
39-47876 1 month ago |
50-71205 50 days |
26935 |
Paul-Lez author:Paul-Lez |
feat(Analysis/SpecialFunction/NthRoot): definition and basic API of Real.nthRoot |
This PR continues the work from #25364.
Original PR: https://github.com/leanprover-community/mathlib4/pull/25364
Co-authored-by: Eric Wieser |
t-analysis |
311/0 |
Mathlib/Analysis/SpecialFunctions/NthRoot.lean |
1 |
10 |
['Paul-Lez', 'eric-wieser', 'github-actions', 'mo271', 'smmercuri', 'yury-harmonic'] |
nobody |
9-40979 9 days ago |
65-76053 2 months ago |
65-76104 65 days |
27313 |
pechersky author:pechersky |
feat(RingTheory/ValuativeRel/Trivial): the trivial valuative relation |
lemmas stated using `[Valuation.Compatible (1 : Valuation R Γ₀)]`
---
[](https://gitpod.io/from-referrer/)
- [x] depends on: #27312
- [x] depends on #28890
|
t-algebra
t-number-theory
label:t-algebra$ |
99/0 |
Mathlib.lean,Mathlib/RingTheory/Valuation/ValuativeRel/Basic.lean,Mathlib/RingTheory/Valuation/ValuativeRel/Trivial.lean |
3 |
12 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
riccardobrasca assignee:riccardobrasca |
9-34925 9 days ago |
16-54869 16 days ago |
25-36154 25 days |
28831 |
qawbecrdtey author:qawbecrdtey |
feat(Logic/Equiv/List): add `decodeList_encodeList_eq_self` and removed unnecessary linter options |
---
This is useful when we call `encode` and `decode` of a list to define a new `Encoder` involving `List`s.
```lean
theorem decodeList_encodeList_eq_self (l : List α) : decodeList (encodeList l) = some l
```
[](https://gitpod.io/from-referrer/)
|
t-logic |
7/6 |
Mathlib/Logic/Equiv/List.lean |
1 |
1 |
['github-actions'] |
awainverse assignee:awainverse |
9-34923 9 days ago |
20-28967 20 days ago |
20-29006 20 days |
28906 |
gasparattila author:gasparattila |
feat(Topology/Algebra/Module): `prod` and `coprod` as `ContinuousLinearEquiv`s |
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-topology
|
36/5 |
Mathlib/Topology/Algebra/Module/LinearMapPiProd.lean,Mathlib/Topology/Algebra/Module/StrongTopology.lean |
2 |
1 |
['github-actions'] |
jcommelin assignee:jcommelin |
9-34922 9 days ago |
18-61489 18 days ago |
18-61527 18 days |
29120 |
eric-wieser author:eric-wieser |
feat: add a typeclass for the indiscrete topology |
Notably, this changes the assumptions of `theorem ContinuousLinearMap.norm_id : ‖id 𝕜 E‖ = 1` from `[NormedAddCommGroup E] [Nontrivial E]` to the more general `[SeminormedAddCommGroup E] [NontrivialTopology E]`.
I've skipped the deprecations since #28102 hasn't made it to any release yet.
As discussed in [#Is there code for X? > Typeclass for nontrivial topology @ 💬](https://leanprover.zulipchat.com/#narrow/channel/217875-Is-there-code-for-X.3F/topic/Typeclass.20for.20nontrivial.20topology/near/533192558) and [#Is there code for X? > Typeclass for indiscrete topology @ 💬](https://leanprover.zulipchat.com/#narrow/channel/217875-Is-there-code-for-X.3F/topic/Typeclass.20for.20indiscrete.20topology/near/512174181)
---
[](https://gitpod.io/from-referrer/)
|
t-topology |
250/76 |
Mathlib/Analysis/Normed/Group/Basic.lean,Mathlib/Analysis/Normed/Group/Hom.lean,Mathlib/Analysis/Normed/Group/SeparationQuotient.lean,Mathlib/Analysis/Normed/Module/RCLike/Real.lean,Mathlib/Analysis/Normed/Operator/Basic.lean,Mathlib/Analysis/Normed/Operator/NormedSpace.lean,Mathlib/Analysis/NormedSpace/Multilinear/Basic.lean,Mathlib/Topology/EMetricSpace/Basic.lean,Mathlib/Topology/Homeomorph/Defs.lean,Mathlib/Topology/Inseparable.lean,Mathlib/Topology/Maps/Basic.lean,Mathlib/Topology/Order.lean,Mathlib/Topology/Sets/Opens.lean,Mathlib/Topology/Sheaves/PUnit.lean |
14 |
4 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
9-32510 9 days ago |
9-41809 9 days ago |
14-26248 14 days |
29328 |
vlad902 author:vlad902 |
feat(SimpleGraph): graph isomorphism preserves `IsAcyclic`/`IsTree` |
---
[](https://gitpod.io/from-referrer/)
|
t-combinatorics |
21/2 |
Mathlib/Combinatorics/SimpleGraph/Acyclic.lean |
1 |
2 |
['github-actions', 'themathqueen'] |
nobody |
9-17853 9 days ago |
9-53339 9 days ago |
9-53364 9 days |
26790 |
FlAmmmmING author:FlAmmmmING |
feat(Combinatorics/Enumerative/Bell.lean): define standard Bell number |
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-combinatorics
|
46/1 |
Mathlib/Combinatorics/Enumerative/Bell.lean |
1 |
11 |
['AntoineChambert-Loir', 'FlAmmmmING', 'eric-wieser', 'github-actions', 'kckennylau', 'madvorak'] |
awainverse assignee:awainverse |
9-17192 9 days ago |
69-66718 2 months ago |
69-66761 69 days |
26986 |
WangYiran01 author:WangYiran01 |
feat(Partition): add bijection for partitions with max part ≤ r |
## Summary
This PR adds a new theorem `partition_max_equals_bound` to `Mathlib.Combinatorics.Enumerative.Partition`.
It constructs a bijection between:
- The set of partitions of `n` in which `r ∈ π.parts` and all parts are `≤ r`, and
- The set of partitions of `n - r` whose largest part is at most `r`.
This provides a constructive proof via removing/adding `r` from/to the partition multiset, in line with classical enumerative combinatorics.
## Implementation notes
- The proof uses `Multiset.erase` and `Multiset.cons` with basic properties of `sum`, `sup`, and `Partition` structures.
- The bijection is implemented explicitly via `f` and `g`, and proven mutually inverse via `Subtype.ext`.
## Linting
- [x] Passes `lake build`
- [x] Linter clean (no commandStart or longLine issues)
## Author
Contributed by Yiran Wang.
|
new-contributor
t-combinatorics
|
85/0 |
Mathlib/Combinatorics/Enumerative/Partition.lean |
1 |
3 |
['WangYiran01', 'github-actions'] |
b-mehta assignee:b-mehta |
9-13726 9 days ago |
64-4878 2 months ago |
64-4919 64 days |
29339 |
kim-em author:kim-em |
feat: add linter for deprecations on different dates not separated by a blank line |
Written by claude. Seems to behave correctly, but I have no opinion on the implementation. I can't work out how to test the behaviour using `#guard_msgs`, however. |
t-linter |
198/0 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter/DeprecatedDates.lean,MathlibTest/Linter/DeprecatedDates.lean |
4 |
8 |
['adomani', 'github-actions'] |
nobody |
9-12289 9 days ago |
9-22350 9 days ago |
9-22393 9 days |
29307 |
harahu author:harahu |
doc: hyphenate attributive compound adjectives ending in "exact" |
Compound adjectives that are attributive (coming before their noun) should almost always be hyphenated in English.
This PR covers such adjectives that are ending in "exact".
---
[](https://gitpod.io/from-referrer/)
|
|
144/144 |
Mathlib/Algebra/Category/ContinuousCohomology/Basic.lean,Mathlib/Algebra/Category/ModuleCat/Free.lean,Mathlib/Algebra/Homology/ConcreteCategory.lean,Mathlib/Algebra/Homology/DerivedCategory/Basic.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/ExactSequences.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/ExtClass.lean,Mathlib/Algebra/Homology/DerivedCategory/HomologySequence.lean,Mathlib/Algebra/Homology/DerivedCategory/ShortExact.lean,Mathlib/Algebra/Homology/DerivedCategory/SingleTriangle.lean,Mathlib/Algebra/Homology/HomologySequence.lean,Mathlib/Algebra/Homology/HomologySequenceLemmas.lean,Mathlib/Algebra/Homology/HomotopyCategory/DegreewiseSplit.lean,Mathlib/Algebra/Homology/HomotopyCategory/HomologicalFunctor.lean,Mathlib/Algebra/Homology/HomotopyCategory/Pretriangulated.lean,Mathlib/Algebra/Homology/HomotopyCategory/ShortExact.lean,Mathlib/Algebra/Homology/LocalCohomology.lean,Mathlib/Algebra/Homology/ShortComplex/ExactFunctor.lean,Mathlib/Algebra/Homology/ShortComplex/ShortExact.lean,Mathlib/Algebra/Lie/Extension.lean,Mathlib/CategoryTheory/Abelian/DiagramLemmas/KernelCokernelComp.lean,Mathlib/CategoryTheory/Abelian/GrothendieckAxioms/Basic.lean,Mathlib/CategoryTheory/Abelian/GrothendieckCategory/ModuleEmbedding/GabrielPopescu.lean,Mathlib/CategoryTheory/Functor/Flat.lean,Mathlib/CategoryTheory/Limits/ExactFunctor.lean,Mathlib/CategoryTheory/Limits/Preserves/Finite.lean,Mathlib/CategoryTheory/Limits/Preserves/Presheaf.lean,Mathlib/CategoryTheory/ObjectProperty/Extensions.lean,Mathlib/CategoryTheory/Preadditive/AdditiveFunctor.lean,Mathlib/CategoryTheory/Preadditive/LeftExact.lean,Mathlib/CategoryTheory/Shift/ShiftSequence.lean,Mathlib/CategoryTheory/Sites/Grothendieck.lean,Mathlib/CategoryTheory/Sites/LeftExact.lean,Mathlib/CategoryTheory/Sites/MayerVietorisSquare.lean,Mathlib/CategoryTheory/Sites/NonabelianCohomology/H1.lean,Mathlib/CategoryTheory/Sites/Sheafification.lean,Mathlib/CategoryTheory/Triangulated/HomologicalFunctor.lean,Mathlib/GroupTheory/GroupExtension/Defs.lean,Mathlib/GroupTheory/MonoidLocalization/GrothendieckGroup.lean,Mathlib/LinearAlgebra/TensorProduct/RightExactness.lean,Mathlib/RepresentationTheory/Coinvariants.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/LongExactSequence.lean,Mathlib/RepresentationTheory/Homological/GroupHomology/LongExactSequence.lean,Mathlib/RingTheory/DedekindDomain/SelmerGroup.lean,Mathlib/RingTheory/Flat/CategoryTheory.lean,Mathlib/RingTheory/Ideal/AssociatedPrime/Finiteness.lean,Mathlib/RingTheory/Regular/IsSMulRegular.lean,Mathlib/Topology/Category/Profinite/Nobeling/Successor.lean |
47 |
n/a |
['github-actions'] |
nobody |
9-11393 9 days ago |
unknown |
unknown |
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/)
|
t-algebra label:t-algebra$ |
192/8 |
Mathlib/RingTheory/DedekindDomain/Different.lean,Mathlib/RingTheory/DedekindDomain/IntegralClosure.lean,Mathlib/RingTheory/FractionalIdeal/Extended.lean,Mathlib/RingTheory/Localization/Basic.lean |
4 |
15 |
['erdOne', 'github-actions', 'mathlib4-merge-conflict-bot', 'xroblot'] |
Vierkantor assignee:Vierkantor |
9-9763 9 days ago |
9-9771 9 days ago |
81-16624 81 days |
27254 |
yuanyi-350 author:yuanyi-350 |
2025 imo problem3 |
- [x] depends on: #28788
- [x] depends on: #28790
- [x] depends on: #28829
---
[](https://gitpod.io/from-referrer/)
|
IMO |
231/0 |
Archive.lean,Archive/Imo/Imo2025Q3.lean,Mathlib/NumberTheory/Padics/PadicVal/Basic.lean |
3 |
28 |
['github-actions', 'jsm28', 'kbuzzard', 'leanprover-community-bot-assistant', 'madvorak', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'themathqueen', 'wwylele', 'yuanyi-350'] |
jsm28 assignee:jsm28 |
9-1341 9 days ago |
10-37007 10 days ago |
44-11875 44 days |
26192 |
kckennylau author:kckennylau |
feat(LinearAlgebra): symmetric tensor power |
This file defines the symmetric tensor power of a module over a ring. The finite powers will form a grading of the symmetric algebra. The n-th symmetric R-tensor power of M will also correspond to global sections of a line bundle on Proj(M) of degree n. It also has a universal property where maps out of it correspond to symmetric multilinear forms.
---
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$ |
137/0 |
Mathlib.lean,Mathlib/LinearAlgebra/TensorPower/Symmetric.lean |
2 |
13 |
['AntoineChambert-Loir', 'erdOne', 'eric-wieser', 'github-actions', 'kckennylau', 'mattrobball'] |
riccardobrasca assignee:riccardobrasca |
8-76327 8 days ago |
33-11214 1 month ago |
82-46386 82 days |
26310 |
kckennylau author:kckennylau |
Binary form |
This PR provides the basic definition of binary forms, which are homogeneous polynomials in two variables.
---
- [ ] depends on: #26312
- [ ] depends on: #26313
- [ ] depends on: #26314
[](https://gitpod.io/from-referrer/)
|
t-algebra
awaiting-author
label:t-algebra$ |
73/0 |
Mathlib.lean,Mathlib/RingTheory/MvPolynomial/BinaryForm.lean |
2 |
13 |
['MichaelStollBayreuth', 'github-actions', 'kckennylau', 'mathlib4-dependent-issues-bot', 'ocfnash'] |
ocfnash assignee:ocfnash |
8-76122 8 days ago |
24-65793 24 days ago |
57-1104 57 days |
27321 |
kckennylau author:kckennylau |
feat(CategoryTheory): Colimit can be computed fiberwise |
We consider category `J` equipped with a functor `F : J ⥤ D` to a discrete category `D`. Then the colimit of any diagram `diagram : J ⥤ C` can be computed using the following algorithm:
1. For each `d : D`, compute the colimit of the restricted diagram `F.fiberIncl d ⋙ diagram`.
2. Take the coproduct of these colimits over all `d : D`.
We call this "computing the colimit fiberwise".
---
Zulip: [#Is there code for X? > over category via a functor](https://leanprover.zulipchat.com/#narrow/channel/217875-Is-there-code-for-X.3F/topic/over.20category.20via.20a.20functor/with/529574191)
[](https://gitpod.io/from-referrer/)
|
t-category-theory
awaiting-CI
|
136/0 |
Mathlib.lean,Mathlib/CategoryTheory/FiberedCategory/Fiber.lean,Mathlib/CategoryTheory/Limits/Shapes/Fiberwise.lean |
3 |
24 |
['github-actions', 'kckennylau', 'robin-carlier'] |
nobody |
8-74005 8 days ago |
8-74005 8 days ago |
19-15685 19 days |
29108 |
JonBannon author:JonBannon |
feat(MeasureTheory): add `LInfty.lean` with `Mul` and `const` related results. |
Continuing to develop pieces needed for a `CStarAlgebra` instance for `Lp R ∞ μ`, we introduce a file `MeasureTheory.Function.LInfty.lean` that takes `MeasureTheory.Function.LpSpace.Basic` and `MeasureTheory.Function.Holder` as imports, and introduces the `Mul` instance on Linfty, and const-related results. In a future PR we will handle `One`, as this will require dealing with `AEEqFun` as well as `Lp` level objects and it's probably best to handle these together in a single PR. We opted to add this file to keep imports light, since adding the `Mul` results to `Basic` would require importing `Holder`, and including these results in `Holder` seemed too specific and would make `Holder` heavier.
---
[](https://gitpod.io/from-referrer/)
|
t-measure-probability
awaiting-author
|
91/0 |
Mathlib.lean,Mathlib/MeasureTheory/Function/LInfty.lean |
2 |
5 |
['JonBannon', 'github-actions', 'j-loreaux'] |
nobody |
8-69006 8 days ago |
10-61670 10 days ago |
4-12126 4 days |
29332 |
Ruben-VandeVelde author:Ruben-VandeVelde |
feat: Set.codRestrict_range_surjective |
---
[](https://gitpod.io/from-referrer/)
|
FLT
t-data
|
5/0 |
Mathlib/Data/Set/Restrict.lean |
1 |
2 |
['github-actions', 'plp127', 'themathqueen'] |
nobody |
8-67261 8 days ago |
8-67551 8 days ago |
9-47978 9 days |
28561 |
euprunin author:euprunin |
chore(Data): golf entire `equivFunOnFintype_single`, `predAbove_right_zero`, `snoc_zero` and more using `rfl` |
---
[](https://gitpod.io/from-referrer/)
|
t-data |
25/88 |
Mathlib/Data/DFinsupp/Defs.lean,Mathlib/Data/Fin/Tuple/Basic.lean,Mathlib/Data/Fin/Tuple/Take.lean,Mathlib/Data/Finmap.lean,Mathlib/Data/Finsupp/AList.lean,Mathlib/Data/Finsupp/Single.lean,Mathlib/Data/Matrix/Basic.lean,Mathlib/Data/Matrix/Block.lean,Mathlib/Data/PFunctor/Multivariate/W.lean,Mathlib/Data/PFunctor/Univariate/M.lean,Mathlib/Data/QPF/Multivariate/Constructions/Cofix.lean,Mathlib/Data/Seq/Computation.lean,Mathlib/Data/Set/Piecewise.lean,Mathlib/Data/Set/Sups.lean,Mathlib/Data/TypeVec.lean,Mathlib/Data/Vector/Basic.lean,Mathlib/Data/Vector/Defs.lean |
17 |
7 |
['github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
8-57739 8 days ago |
8-57763 8 days ago |
24-32994 24 days |
29321 |
FormulaRabbit81 author:FormulaRabbit81 |
feat(Topology): obtain new distance structures on pseudo(e)metricspaces |
---
[](https://gitpod.io/from-referrer/)
|
t-topology
awaiting-CI
WIP
|
130/65 |
Mathlib/Analysis/Normed/Lp/PiLp.lean,Mathlib/Analysis/Normed/Lp/ProdLp.lean,Mathlib/Topology/MetricSpace/Basic.lean,Mathlib/Topology/MetricSpace/PiNat.lean,Mathlib/Topology/MetricSpace/Pseudo/Constructions.lean,Mathlib/Topology/MetricSpace/Pseudo/Defs.lean,Mathlib/Topology/MetricSpace/Pseudo/Pi.lean,Mathlib/Topology/MetricSpace/UniformConvergence.lean |
8 |
7 |
['FormulaRabbit81', 'YaelDillies', 'github-actions'] |
nobody |
8-41941 8 days ago |
8-41941 8 days ago |
0-76797 21 hours |
22954 |
eric-wieser author:eric-wieser |
feat(RingTheory/Congruence/Hom): copy from GroupTheory |
This was motivated in review of #22355, but I no longer recall why.
It also helps with #29357.
Either way, this captures a definition that was inlined in a later file.
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory |
214/16 |
Mathlib/Algebra/RingQuot.lean,Mathlib/GroupTheory/Congruence/Hom.lean,Mathlib/RingTheory/Congruence/Defs.lean,Mathlib/RingTheory/Congruence/Hom.lean,Mathlib/RingTheory/TwoSidedIdeal/Kernel.lean |
5 |
2 |
['github-actions', 'leanprover-community-bot-assistant'] |
nobody |
8-36846 8 days ago |
8-36868 8 days ago |
120-5734 120 days |
25843 |
mitchell-horner author:mitchell-horner |
feat(Combinatorics/SimpleGraph): define `between` subgraphs |
The simple graph `G.between s t` is the subgraph of `G` containing edges that connect a vertex in the set `s` to a vertex in the set `t`.
---
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #24948.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/24948* |
t-combinatorics |
86/0 |
Mathlib/Combinatorics/SimpleGraph/Bipartite.lean |
1 |
1 |
['github-actions'] |
b-mehta assignee:b-mehta |
8-34919 8 days ago |
91-75668 2 months ago |
91-75649 91 days |
27178 |
artie2000 author:artie2000 |
feat(Algebra/Order/Ring): make `IsOrderedRing.toStrictOrderedRing` an instance |
Requiring `IsStrictOrderedRing` on a `Field` is a footgun (the current instances come from a find and replace on `LinearOrderedField`). Weakening typeclasses can incur a performance hit so will be done where appropriate in future PRs.
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
RFC
|
2/1 |
Mathlib/Algebra/Order/Ring/Defs.lean |
1 |
22 |
['YaelDillies', 'alreadydone', 'artie2000', 'eric-wieser', 'github-actions', 'j-loreaux', 'leanprover-bot', 'leanprover-community-mathlib4-bot'] |
erdOne assignee:erdOne |
8-34918 8 days ago |
16-32319 16 days ago |
29-37730 29 days |
29027 |
grunweg author:grunweg |
feat/fix(FlexibleLinter): mark more tactics as flexible |
and add proper tests for all of these. In particular, this PR
- fixes the handling of `(n)linarith` (which had a bug), and adds a test,
- adds `ring!` and `abel!` (as flexible tactics),
- adds `ring_nf!` and `abel_nf!` as stopper tactics,
- adds `cfc_tac` and its sisters as flexible tactic (as they use aesop and/or fun_prop),
- adds `continuity` and `measurability` as flexible (as they are aesop-based),
- add `group` and `module` as flexible,
- add `grind` as flexible,
- add `positivity` and `finiteness` as flexible, and `finiteness_nonterminal` as stopper tactic.
I'm happy to discuss any of these particular additions further.
---
Zulip discussion at https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/flexible.20vs.20rigid.20tactics/with/536424236.
[](https://gitpod.io/from-referrer/)
|
t-linter |
232/56 |
Mathlib/Tactic/Linter/FlexibleLinter.lean,MathlibTest/FlexibleLinter.lean,MathlibTest/ImportHeavyFlexibleLinter.lean |
3 |
16 |
['adomani', 'b-mehta', 'github-actions', 'grunweg'] |
joneugster assignee:joneugster |
8-34913 8 days ago |
16-61956 16 days ago |
16-61938 16 days |
27995 |
kckennylau author:kckennylau |
feat(RingTheory/Valuation): alternate constructors for Valuation |
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
awaiting-CI
|
82/0 |
Mathlib/Algebra/GroupWithZero/WithZero.lean,Mathlib/FieldTheory/RatFunc/Degree.lean,Mathlib/NumberTheory/Padics/PadicNumbers.lean,Mathlib/RingTheory/Valuation/Basic.lean |
4 |
22 |
['YaelDillies', 'github-actions', 'grunweg', 'kckennylau', 'pechersky'] |
nobody |
8-12854 8 days ago |
8-12854 8 days ago |
18-47707 18 days |
28546 |
Sfgangloff author:Sfgangloff |
feat(SymbolicDynamics): basic setup of Zd, full shift, cylinders, pat… |
# Symbolic dynamics on groups: core API and entropy along finite shapes
This PR adds a **group-generic** foundation for symbolic dynamics over an arbitrary group `G`, together with convenient specializations for `ℤ` and `ℤ^d`.
## Summary of additions
- **Full shift and shift action**
- `abbrev FullShift (A G) := G → A` (inherits product topology from the Π-type).
- Right shift `shift g x` with convention `(shift g x) h = x (h * g)`.
- **Cylinders and topology**
- `cylinder U x : Set (G → A)` for finite `U : Finset G`.
- Cylinders are open under `[DiscreteTopology A]`; with a finite alphabet they are also closed.
- Equality with dependent products:
`cylinder U x = Set.pi (↑U) (fun i => ({x i} : Set A))`, enabling use of the `Set.pi` API.
- **Patterns, occurrences, and subshifts**
- `Pattern A G` with finite `support : Finset G` and `data : support → A`.
- `Pattern.occursIn p x g` (occurrence at translate `g`) and the expected shift law.
- `forbids F` and `Subshift A G` (closed, shift-invariant subsets).
- `FixedSupport A G U` with an equivalence to `(U → A)` to obtain finiteness.
- **Language on finite shapes and counting**
- `languageOn X U`, `languageCardOn X U`, and `patternCountOn Y U`.
- **Entropy along a shape sequence**
- `limsupAtTop` (as an `sInf` of eventual upper bounds).
- `entropyAlong X F hF := limsup (log (patternCountOn X (F n) + 1) / |F n|)`
for any nonempty finite shapes `F : ℕ → Finset G` (the `+ 1` avoids `log 0`).
- **Specializations**
- `IntShapes`: segments `[-n,n]` on `Multiplicative ℤ`, with `entropy_Z`.
- `ZdShapes`: boxes `[-n,n]^d` on `ℤ^d` (as functions `Fin d → ℤ`), with `entropy_Zd`.
## Mathematical remarks
- The API is **shape-parametric**: entropy is defined along user-provided finite shapes.
- On **amenable** groups, using a **Følner** sequence yields a canonical value (Ornstein–Weiss).
This PR does not assume amenability; the family of shapes is an explicit input.
## Motivation
Provide a clean, reusable base for symbolic dynamics on groups in mathlib.
## Future work
- Add a Følner predicate and prove shape-independence / limit existence on amenable groups.
- Expand the `ℤ`/`ℤ^d` toolkit (alternative shapes, mixing, factors).
- Develop 1D theory and, longer-term, multidimensional SFT results (e.g. along the lines of Hochman–Meyerovitch).
|
new-contributor
t-dynamics
|
513/0 |
Mathlib.lean,Mathlib/Dynamics/SymbolicDynamics/Basic.lean,Mathlib/Dynamics/SymbolicDynamics/EntropyFinitelyGenerated.lean |
3 |
14 |
['Sfgangloff', 'eric-wieser', 'github-actions', 'kckennylau', 'sgouezel'] |
sgouezel assignee:sgouezel |
8-11627 8 days ago |
26-76698 26 days ago |
26-76737 26 days |
26277 |
AntoineChambert-Loir author:AntoineChambert-Loir |
feat(RingTheory/Congruence/Hom): prove basic isomorphisms theorems for ring congruences |
This file contains elementary definitions involving congruence
relations and morphisms for semirings, rings, and algebras.
* `RingCon.ker`: the kernel of a monoid homomorphism as a congruence relation
* `RingCon.lift`, `RingCon.liftₐ`: the homomorphism / the algebra morphism
on the quotient given that the congruence is in the kernel
* `RingCon.map`, `RingCon.mapₐ`: homomorphism / algebra morphism
from a smaller to a larger quotient
* `RingCon.quotientKerEquivRangeS`, `RingCon.quotientKerEquivRange`,
`RingCon.quotientKerEquivRangeₐ` :
the first isomorphism theorem for semirings (using `RingHom.rangeS`),
rings (using `RingHom.range`) and algebras (using `AlgHom.range`).
* `RingCon.comapQuotientEquivRangeS`, `RingCon.comapQuotientEquivRange`,
`RingCon.comapQuotientEquivRangeₐ` : the second isomorphism theorem
for semirings (using `RingHom.rangeS`), rings (using `RingHom.range`)
and algebras (using `AlgHom.range`).
* `RingCon.quotientQuotientEquivQuotient`, `RingCon.quotientQuotientEquivQuotientₐ` :
the third isomorphism theorem for semirings (or rings) and algebras
It is an adaptation of what existed for multiplicative congruences (docs#Con) and is only useful for semirings which are not rings.
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory |
554/2 |
Mathlib.lean,Mathlib/Algebra/Ring/Subsemiring/Basic.lean,Mathlib/Algebra/RingQuot.lean,Mathlib/RingTheory/Congruence/Defs.lean,Mathlib/RingTheory/Congruence/Hom.lean |
5 |
4 |
['AntoineChambert-Loir', 'eric-wieser', 'github-actions'] |
joneugster assignee:joneugster |
8-11573 8 days ago |
39-3959 1 month ago |
82-46578 82 days |
28613 |
espottesmith author:espottesmith |
feat(Combinatorics): define undirected hypergraphs |
This PR defines undirected hypergraphs:
```
@[ext]
structure Hypergraph (α : Type*) where
/-- The vertex set -/
vertexSet : Set α
/-- The hyperedge set -/
hyperedgeSet : Set (Set α)
/-- All hyperedges must be subsets of the vertex set -/
hyperedge_isSubset_vertexSet : ∀ ⦃e⦄, e ∈ hyperedgeSet → e ⊆ vertexSet
```
In addition to the main definition, some additional definitions and related lemmas are provided:
- vertex adjacency
- hyperedge adjacency
- vertex "stars"
- special cases (loops, empty hypergraphs, trivial hypergraphs, complete hypergraphs, simple hypergraphs, k-uniform hypergraphs, and d-regular hypergraphs)
- (some) hypergraph cardinality
- subhypergraphs, induced subhypergraphs, and partial hypergraphs
This implementation is certainly bare-bones. I'm submitting this PR at this point, rather than when my developments are more fleshed out, because there has been some interest in others contributing to hypergraph formalization in mathlib.
In the near future, goals include:
- defining incidence matrices (i.e., conversion from `Hypergraph α` to `Matrix α (Set α) β`
- coersion/generalization of graph as 2-uniform hypergraph
- conversion of a hypergraph into its associated clique graph/two-section graph
- constructing the dual of a hypergraph (note: on first blush, this appears somewhat challenging, given that we define hyperedges as `Set α` rather than some other type `β`)
- rank and co-rank
- walks, paths, cycles, etc. on hypergraphs
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-combinatorics
|
375/0 |
Mathlib.lean,Mathlib/Combinatorics/Hypergraph/Basic.lean |
2 |
52 |
['b-mehta', 'espottesmith', 'github-actions', 'jt496', 'lauramonk', 'mathlib4-merge-conflict-bot'] |
b-mehta assignee:b-mehta |
8-969 8 days ago |
8-969 8 days ago |
13-73556 13 days |
29356 |
Paul-Lez author:Paul-Lez |
feat(Mathlib/FieldTheory/RatFunc/Basic): add characteristic instances for `RatFunc` |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
55/9 |
Mathlib/Algebra/Algebra/Basic.lean,Mathlib/Algebra/Algebra/Field.lean,Mathlib/Algebra/Algebra/IsSimpleRing.lean,Mathlib/Algebra/CharP/Algebra.lean,Mathlib/Analysis/RCLike/Basic.lean,Mathlib/FieldTheory/RatFunc/Basic.lean |
6 |
7 |
['eric-wieser', 'github-actions'] |
nobody |
7-84733 7 days ago |
8-44770 8 days ago |
8-44805 8 days |
29028 |
themathqueen author:themathqueen |
feat(Algebra/Star): define `unitary R →* StarAlgEquiv S R R` |
Every unitary defines a star-algebra automorphism (this is an extension of a special version of `MulSemiringAction.toRingEquiv` for unitaries).
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
64/0 |
Mathlib.lean,Mathlib/Algebra/Star/UnitaryStarAlgAut.lean |
2 |
14 |
['eric-wieser', 'github-actions', 'themathqueen'] |
eric-wieser assignee:eric-wieser |
7-65965 7 days ago |
15-3454 15 days ago |
16-60464 16 days |
28836 |
yury-harmonic author:yury-harmonic |
feat: add `norm_num` extensions |
Add `norm_num` extensions for
- `Int.negOfNat`;
- `Nat.floor`, `Nat.ceil`, `Int.fract`, and `Int.round`.
---
[](https://gitpod.io/from-referrer/)
|
t-meta
awaiting-author
|
319/7 |
Mathlib/Algebra/Order/Floor/Semiring.lean,Mathlib/Data/NNRat/Floor.lean,Mathlib/Data/Rat/Floor.lean,Mathlib/Tactic/NormNum/Basic.lean,MathlibTest/norm_num_ext.lean |
5 |
8 |
['Ruben-VandeVelde', 'digama0', 'eric-wieser', 'github-actions'] |
j-loreaux assignee:j-loreaux |
7-64813 7 days ago |
7-64813 7 days ago |
12-38307 12 days |
26339 |
mans0954 author:mans0954 |
feat(Analysis/Normed/Module/WeakDual): Banach Dieudonné Lemma |
This PR continues the work from #16316.
Original PR: https://github.com/leanprover-community/mathlib4/pull/16316 |
large-import
t-analysis
WIP
|
377/3 |
Mathlib/Analysis/LocallyConvex/AbsConvex.lean,Mathlib/Analysis/LocallyConvex/Polar.lean,Mathlib/Analysis/Normed/Module/WeakDual.lean,Mathlib/Topology/UniformSpace/Cauchy.lean |
4 |
n/a |
['github-actions', 'mans0954', 'mathlib4-merge-conflict-bot'] |
nobody |
7-60850 7 days ago |
unknown |
unknown |
29355 |
girving author:girving |
feat(Trigonometric): Taylor series bounds for sin and cos |
Zulip discussion here:
https://leanprover.zulipchat.com/#narrow/channel/217875-Is-there-code-for-X.3F/topic/Better.20.60Real.2Esin.60.20bounds/near/535035576
We also include the full set of intervals on which sin and cos are monotone/antitone.
---
Questions to resolve as part of review:
1. I've left the `Finset.sum_range_even` in the new `SeriesBounds` file, but presumably it should go somewhere else (unless you want me to inline it, but that seems worse).
2. Is putting the new Taylor series bounds in a new `SeriesBounds` file right, or should it go in the current `Bounds.lean` file? When I started writing the PR I thought the new bounds would need more imports via more analysis, but it turns out the only new import needed would be `Mathlib.Algebra.BigOperators.Field` which seems lightweight. I am happy with whatever the preference is in terms of file structure.
[](https://gitpod.io/from-referrer/)
|
t-analysis |
158/0 |
Mathlib.lean,Mathlib/Algebra/BigOperators/Ring/Finset.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Bounds.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/SeriesBounds.lean |
4 |
24 |
['Parcly-Taxel', 'Ruben-VandeVelde', 'girving', 'github-actions', 'llllvvuu'] |
nobody |
7-55666 7 days ago |
8-43891 8 days ago |
8-49773 8 days |
19046 |
j-loreaux author:j-loreaux |
feat: define class `SemigroupAction` |
---
If I can get this building with minimal performance impact, I would like to change the names to:
`MulAction → MonoidAction`
`SemigroupAction → MulAction`
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
48/26 |
Mathlib/Algebra/Azumaya/Matrix.lean,Mathlib/Algebra/Category/ModuleCat/Presheaf.lean,Mathlib/Algebra/Group/Action/Defs.lean,Mathlib/Algebra/Group/Action/Hom.lean,Mathlib/Algebra/Group/Action/Prod.lean,Mathlib/Algebra/Group/Action/TypeTags.lean,Mathlib/Algebra/Polynomial/Laurent.lean,Mathlib/GroupTheory/CoprodI.lean,Mathlib/LinearAlgebra/Eigenspace/Matrix.lean,Mathlib/LinearAlgebra/FreeModule/Finite/Quotient.lean,Mathlib/LinearAlgebra/Matrix/SesquilinearForm.lean,Mathlib/NumberTheory/ModularForms/CongruenceSubgroups.lean,Mathlib/RingTheory/Trace/Basic.lean |
13 |
10 |
['alreadydone', 'github-actions', 'j-loreaux', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'urkud'] |
jcommelin assignee:jcommelin |
7-34925 7 days ago |
15-51155 15 days ago |
21-78446 21 days |
28311 |
eric-wieser author:eric-wieser |
fix(Tactic/NormNum): do not hang on large powers |
This uses `Lean.checkExponent` to guard against large powers.
Unfortunately the log messages it emits are currently swallowed, but surfacing these may require changing the API for norm_num extensions (to live in `OptionT MetaM`) and so is left to future work.
---
[](https://gitpod.io/from-referrer/)
|
t-meta
bug
|
41/23 |
Mathlib/Tactic/NormNum/Pow.lean,Mathlib/Tactic/Ring/Basic.lean,MathlibTest/norm_num.lean,MathlibTest/norm_num_ext.lean |
4 |
4 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
robertylewis assignee:robertylewis |
7-34923 7 days ago |
16-41579 16 days ago |
24-8398 24 days |
28858 |
themathqueen author:themathqueen |
feat(LinearAlgebra/Matrix/PosDef): inner product on matrices induced by positive definite matrix |
This defines an inner product on matrices induced by a positive definite matrix `M`: `inner x y = trace (M * xᴴ * y)`. When `M = 1`, this is exactly the [Frobenius inner product](https://en.wikipedia.org/wiki/Frobenius_inner_product).
---
- [x] depends on: #28773
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
29/0 |
Mathlib/LinearAlgebra/Matrix/PosDef.lean |
1 |
8 |
['eric-wieser', 'github-actions', 'mathlib4-dependent-issues-bot', 'themathqueen'] |
riccardobrasca assignee:riccardobrasca |
7-34921 7 days ago |
14-56187 14 days ago |
14-57657 14 days |
29040 |
PMKielstra author:PMKielstra |
feat: trapezoidal rule for integration |
This PR defines the trapezoidal rule and proves the standard error bound on it in terms of bounds on the second derivative.
I have vague plans of using this plus interval arithmetic to develop a tactic that can automatically close goals of the form `\integral x in a..b, f x < y` or similar.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-measure-probability
|
273/0 |
Mathlib.lean,Mathlib/MeasureTheory/Integral/IntervalIntegral/Basic.lean,Mathlib/MeasureTheory/Integral/IntervalIntegral/TrapezoidalRule.lean |
3 |
40 |
['PMKielstra', 'github-actions', 'tb65536'] |
kex-y assignee:kex-y |
7-34919 7 days ago |
16-41812 16 days ago |
16-42254 16 days |
29042 |
vihdzp author:vihdzp |
feat(SetTheory/Ordinal/Exponential): generalize theorems from `y = succ x` to `x < y` |
---
[](https://gitpod.io/from-referrer/)
|
t-set-theory |
18/6 |
Mathlib/SetTheory/Ordinal/Exponential.lean |
1 |
1 |
['github-actions'] |
b-mehta assignee:b-mehta |
7-34918 7 days ago |
16-31560 16 days ago |
16-31549 16 days |
29058 |
vihdzp author:vihdzp |
feat: `Colex` type synonym |
We create a new `Colex` type synonym for the colexicographic order on a type. We use this to re-define the colexicographic order on `Finset`, protecting and deprecating the existing `Finset.Colex` type synonym.
A future PR will add instances for `Pi` types and `Finsupp`.
See [Zulip](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Pi.2ELex/near/536563593) for some discussion on this.
---
[](https://gitpod.io/from-referrer/)
|
t-order |
152/59 |
Mathlib/Combinatorics/Colex.lean,Mathlib/Order/Synonym.lean |
2 |
1 |
['github-actions'] |
bryangingechen assignee:bryangingechen |
7-34917 7 days ago |
15-83322 15 days ago |
15-83318 15 days |
29082 |
grunweg author:grunweg |
RFC: tag `IsInducing` and `Is{Open,Closed,}Embedding` with `fun_prop` |
I have not tested if this is usable in practice; perhaps it is not.
---
[](https://gitpod.io/from-referrer/)
|
t-topology |
37/5 |
Mathlib/Topology/Constructions.lean,Mathlib/Topology/Defs/Induced.lean,Mathlib/Topology/Maps/Basic.lean |
3 |
1 |
['github-actions'] |
jcommelin assignee:jcommelin |
7-34916 7 days ago |
15-53568 15 days ago |
15-53604 15 days |
29114 |
jeremypparker author:jeremypparker |
feat(MeasureTheory.Integral): Mean value theorem for integrals |
Combines results from MeasureTheory.Integral.Average and the intermediate value theorem to give the integral form of the mean value theorem: https://en.wikipedia.org/wiki/Mean_value_theorem#Mean_value_theorems_for_definite_integrals
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-measure-probability
|
55/0 |
Mathlib/MeasureTheory/Integral/IntervalAverage.lean |
1 |
1 |
['github-actions'] |
sgouezel assignee:sgouezel |
7-34914 7 days ago |
14-60909 14 days ago |
14-60948 14 days |
29119 |
JovanGerb author:JovanGerb |
fix(Tactic/ToAdditive/Frontend): swap `reorderForall` and `applyReplacementForall` |
This PR does some general clean-up in the `to_additive` implementation:
- `expand` is moved up so that it can be called directly inside of `applyReplacementFun`. The current situation requires uses of `applyReplacementFun` to know that they need to call `expand` first.
- `applyReplacementFun` is significantly cleaned up, without changing the implementation, making it shorter, more readable and more efficient.
- It swaps reorderForall/Lambda with applyReplacementForall/Lambda, because in the previous order, if `reorder` would reorder some argument that appears in `dontTranslate`, it would do the wrong thing (although I don't think this will ever come up in practice)
---
[](https://gitpod.io/from-referrer/)
|
t-meta |
93/106 |
Mathlib/Tactic/ToAdditive/Frontend.lean,MathlibTest/toAdditive.lean |
2 |
1 |
['github-actions'] |
robertylewis assignee:robertylewis |
7-34913 7 days ago |
14-49091 14 days ago |
14-49127 14 days |
27882 |
euprunin author:euprunin |
chore: golf using `grind [Nat.cast_*]` |
|
|
6/18 |
Mathlib/Analysis/SpecialFunctions/Trigonometric/Cotangent.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/EulerSineProd.lean,Mathlib/GroupTheory/CommutingProbability.lean,Mathlib/RingTheory/ZMod/UnitsCyclic.lean |
4 |
10 |
['github-actions', 'kim-em', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'mathlib4-merge-conflict-bot'] |
urkud assignee:urkud |
7-8257 7 days ago |
7-8257 7 days ago |
41-50780 41 days |
27370 |
euprunin author:euprunin |
chore(Tactic/CancelDenoms): golf `cancel_factors_eq` |
---
Show trace profiling of cancel_factors_eq : 120 ms before, 46 ms after 🎉
### Trace profiling of `cancel_factors_eq` before PR 27370
```diff
diff --git a/Mathlib/Tactic/CancelDenoms/Core.lean b/Mathlib/Tactic/CancelDenoms/Core.lean
index c4b62d3e29..3ec2128994 100644
--- a/Mathlib/Tactic/CancelDenoms/Core.lean
+++ b/Mathlib/Tactic/CancelDenoms/Core.lean
@@ -80,6 +80,7 @@ theorem cancel_factors_le {α} [Field α] [LinearOrder α] [IsStrictOrderedRing
· exact mul_pos had hbd
· exact one_div_pos.2 hgcd
+set_option trace.profiler true in
theorem cancel_factors_eq {α} [Field α] {a b ad bd a' b' gcd : α} (ha : ad * a = a')
(hb : bd * b = b') (had : ad ≠ 0) (hbd : bd ≠ 0) (hgcd : gcd ≠ 0) :
(a = b) = (1 / gcd * (bd * a') = 1 / gcd * (ad * b')) := by
```
```
ℹ [436/436] Built Mathlib.Tactic.CancelDenoms.Core (2.8s)
info: Mathlib/Tactic/CancelDenoms/Core.lean:84:0: [Elab.command] [0.015258] theorem cancel_factors_eq {α} [Field α] {a b ad bd a' b' gcd : α} (ha : ad * a = a')
(hb : bd * b = b') (had : ad ≠ 0) (hbd : bd ≠ 0) (hgcd : gcd ≠ 0) :
(a = b) = (1 / gcd * (bd * a') = 1 / gcd * (ad * b')) :=
by
rw [← ha, ← hb, ← mul_assoc bd, ← mul_assoc ad, mul_comm bd]
ext; constructor
· rintro rfl
rfl
· intro h
simp only [← mul_assoc] at h
refine mul_left_cancel₀ (mul_ne_zero ?_ ?_) h
on_goal 1 => apply mul_ne_zero
on_goal 1 => apply div_ne_zero
· exact one_ne_zero
all_goals assumption
[Elab.definition.header] [0.014988] CancelDenoms.cancel_factors_eq
info: Mathlib/Tactic/CancelDenoms/Core.lean:84:0: [Elab.async] [0.122474] elaborating proof of CancelDenoms.cancel_factors_eq
[Elab.definition.value] [0.119890] CancelDenoms.cancel_factors_eq
[Elab.step] [0.118614]
rw [← ha, ← hb, ← mul_assoc bd, ← mul_assoc ad, mul_comm bd]
ext; constructor
· rintro rfl
rfl
· intro h
simp only [← mul_assoc] at h
refine mul_left_cancel₀ (mul_ne_zero ?_ ?_) h
on_goal 1 => apply mul_ne_zero
on_goal 1 => apply div_ne_zero
· exact one_ne_zero
all_goals assumption
[Elab.step] [0.118601]
rw [← ha, ← hb, ← mul_assoc bd, ← mul_assoc ad, mul_comm bd]
ext; constructor
· rintro rfl
rfl
· intro h
simp only [← mul_assoc] at h
refine mul_left_cancel₀ (mul_ne_zero ?_ ?_) h
on_goal 1 => apply mul_ne_zero
on_goal 1 => apply div_ne_zero
· exact one_ne_zero
all_goals assumption
[Elab.step] [0.010324] rw [← ha, ← hb, ← mul_assoc bd, ← mul_assoc ad, mul_comm bd]
[Elab.step] [0.010312] (rewrite [← ha, ← hb, ← mul_assoc bd, ← mul_assoc ad, mul_comm bd];
with_annotate_state"]" (try (with_reducible rfl)))
[Elab.step] [0.010299] rewrite [← ha, ← hb, ← mul_assoc bd, ← mul_assoc ad, mul_comm bd];
with_annotate_state"]" (try (with_reducible rfl))
[Elab.step] [0.010291] rewrite [← ha, ← hb, ← mul_assoc bd, ← mul_assoc ad, mul_comm bd];
with_annotate_state"]" (try (with_reducible rfl))
[Elab.step] [0.105805] ·
intro h
simp only [← mul_assoc] at h
refine mul_left_cancel₀ (mul_ne_zero ?_ ?_) h
on_goal 1 => apply mul_ne_zero
on_goal 1 => apply div_ne_zero
· exact one_ne_zero
all_goals assumption
[Elab.step] [0.105661]
intro h
simp only [← mul_assoc] at h
refine mul_left_cancel₀ (mul_ne_zero ?_ ?_) h
on_goal 1 => apply mul_ne_zero
on_goal 1 => apply div_ne_zero
· exact one_ne_zero
all_goals assumption
[Elab.step] [0.105650]
intro h
simp only [← mul_assoc] at h
refine mul_left_cancel₀ (mul_ne_zero ?_ ?_) h
on_goal 1 => apply mul_ne_zero
on_goal 1 => apply div_ne_zero
· exact one_ne_zero
all_goals assumption
[Elab.step] [0.043946] refine mul_left_cancel₀ (mul_ne_zero ?_ ?_) h
[Elab.step] [0.043859] expected type: a = b, term
mul_left_cancel₀ (mul_ne_zero ?_ ?_) h
[Elab.step] [0.025447] expected type: ?m.103 * ?m.104 ≠ 0, term
(mul_ne_zero ?_ ?_)
[Elab.step] [0.025432] expected type: ?m.103 * ?m.104 ≠ 0, term
mul_ne_zero ?_ ?_
[Meta.synthInstance] [0.019262] ✅️ NoZeroDivisors α
[Elab.step] [0.021441] on_goal 1 => apply mul_ne_zero
[Elab.step] [0.019543] apply mul_ne_zero
[Elab.step] [0.019530] apply mul_ne_zero
[Elab.step] [0.019514] apply mul_ne_zero
[Meta.synthInstance] [0.013986] ✅️ NoZeroDivisors α
[Elab.step] [0.018650] · exact one_ne_zero
[Elab.step] [0.018355] exact one_ne_zero
[Elab.step] [0.018309] exact one_ne_zero
[Elab.step] [0.018269] exact one_ne_zero
[Elab.step] [0.017827] expected type: 1 ≠ 0, term
one_ne_zero
[Meta.synthInstance] [0.012295] ✅️ NeZero 1
Build completed successfully (436 jobs).
```
### Trace profiling of `cancel_factors_eq` after PR 27370
```diff
diff --git a/Mathlib/Tactic/CancelDenoms/Core.lean b/Mathlib/Tactic/CancelDenoms/Core.lean
index c4b62d3e29..066f915189 100644
--- a/Mathlib/Tactic/CancelDenoms/Core.lean
+++ b/Mathlib/Tactic/CancelDenoms/Core.lean
@@ -80,20 +80,11 @@ theorem cancel_factors_le {α} [Field α] [LinearOrder α] [IsStrictOrderedRing
· exact mul_pos had hbd
· exact one_div_pos.2 hgcd
+set_option trace.profiler true in
theorem cancel_factors_eq {α} [Field α] {a b ad bd a' b' gcd : α} (ha : ad * a = a')
(hb : bd * b = b') (had : ad ≠ 0) (hbd : bd ≠ 0) (hgcd : gcd ≠ 0) :
(a = b) = (1 / gcd * (bd * a') = 1 / gcd * (ad * b')) := by
- rw [← ha, ← hb, ← mul_assoc bd, ← mul_assoc ad, mul_comm bd]
- ext; constructor
- · rintro rfl
- rfl
- · intro h
- simp only [← mul_assoc] at h
- refine mul_left_cancel₀ (mul_ne_zero ?_ ?_) h
- on_goal 1 => apply mul_ne_zero
- on_goal 1 => apply div_ne_zero
- · exact one_ne_zero
- all_goals assumption
+ grind
theorem cancel_factors_ne {α} [Field α] {a b ad bd a' b' gcd : α} (ha : ad * a = a')
(hb : bd * b = b') (had : ad ≠ 0) (hbd : bd ≠ 0) (hgcd : gcd ≠ 0) :
```
```
ℹ [436/436] Built Mathlib.Tactic.CancelDenoms.Core (3.1s)
info: Mathlib/Tactic/CancelDenoms/Core.lean:84:0: [Elab.command] [0.034809] theorem cancel_factors_eq {α} [Field α] {a b ad bd a' b' gcd : α} (ha : ad * a = a')
(hb : bd * b = b') (had : ad ≠ 0) (hbd : bd ≠ 0) (hgcd : gcd ≠ 0) :
(a = b) = (1 / gcd * (bd * a') = 1 / gcd * (ad * b')) := by grind
[Elab.definition.header] [0.014091] CancelDenoms.cancel_factors_eq
info: Mathlib/Tactic/CancelDenoms/Core.lean:84:0: [Elab.async] [0.046425] elaborating proof of CancelDenoms.cancel_factors_eq
[Elab.definition.value] [0.045869] CancelDenoms.cancel_factors_eq
[Elab.step] [0.045340] grind
[Elab.step] [0.045327] grind
[Elab.step] [0.045311] grind
info: Mathlib/Tactic/CancelDenoms/Core.lean:87:2: [Elab.async] [0.027621] Lean.addDecl
[Kernel] [0.027585] ✅️ typechecking declarations [CancelDenoms.cancel_factors_eq._proof_1_1]
Build completed successfully (436 jobs).
```
|
t-meta |
1/11 |
Mathlib/Tactic/CancelDenoms/Core.lean |
1 |
7 |
['euprunin', 'github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot'] |
alexjbest assignee:alexjbest |
7-6742 7 days ago |
7-6742 7 days ago |
52-41432 52 days |
27252 |
Parcly-Taxel author:Parcly-Taxel |
feat: sharp bounds for `‖exp (I * x) - 1‖` when `x` is real |
From Carleson |
carleson
t-analysis
|
44/0 |
Mathlib/Analysis/Complex/Trigonometric.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Bounds.lean |
2 |
12 |
['Parcly-Taxel', 'eric-wieser', 'github-actions', 'grunweg', 'mathlib4-merge-conflict-bot'] |
nobody |
6-84572 6 days ago |
7-929 7 days ago |
8-7390 8 days |
29271 |
euprunin author:euprunin |
chore: remove redundant `let` and `letI` invocations |
---
[](https://gitpod.io/from-referrer/)
|
maintainer-merge |
1/8 |
Mathlib/Algebra/Algebra/TransferInstance.lean,Mathlib/Algebra/Module/FinitePresentation.lean,Mathlib/CategoryTheory/Monoidal/Grp_.lean,Mathlib/ModelTheory/Algebra/Ring/FreeCommRing.lean,Mathlib/Topology/Metrizable/Uniformity.lean |
5 |
10 |
['JovanGerb', 'github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'ocfnash'] |
nobody |
6-80976 6 days ago |
6-83508 6 days ago |
10-43089 10 days |
28000 |
daefigueroa author:daefigueroa |
feat(Dynamics/Flow): define semiconjugacy, factor and orbit |
We add definitions relating to flows.
This contribution was created as part of the Utrecht Summerschool "Formalizing Mathematics in Lean" in July 2025.
---
[](https://gitpod.io/from-referrer/) |
new-contributor
t-dynamics
|
116/3 |
Mathlib/Dynamics/Flow.lean |
1 |
7 |
['chrisflav', 'daefigueroa', 'github-actions'] |
nobody |
6-75016 6 days ago |
6-75756 6 days ago |
15-32151 15 days |
29365 |
staroperator author:staroperator |
feat(SetTheory/ZFC): add `ZFSet.card` |
The same as `ZFSet.rank`, we define `ZFSet.card` as `ZFSet.{u} → Cardinal.{u}` and prove some basic properties.
---
[](https://gitpod.io/from-referrer/)
|
t-set-theory |
123/4 |
Mathlib.lean,Mathlib/SetTheory/Cardinal/Basic.lean,Mathlib/SetTheory/ZFC/Basic.lean,Mathlib/SetTheory/ZFC/Cardinal.lean |
4 |
2 |
['github-actions', 'staroperator', 'vihdzp'] |
nobody |
6-74595 6 days ago |
7-81601 7 days ago |
7-81641 7 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
---
[](https://gitpod.io/from-referrer/) |
t-algebra
awaiting-author
label:t-algebra$ |
34/0 |
Mathlib/Algebra/QuadraticDiscriminant.lean |
1 |
8 |
['chrisflav', 'github-actions', 'tb65536', 'upobir'] |
chrisflav assignee:chrisflav |
6-72158 6 days ago |
30-63686 30 days ago |
55-10605 55 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-ring-theory
awaiting-zulip
|
76/8 |
Mathlib/Algebra/Polynomial/Coeff.lean,Mathlib/RingTheory/Polynomial/SmallDegreeVieta.lean |
2 |
44 |
['chrisflav', 'github-actions', 'kckennylau', 'mans0954', 'ocfnash'] |
chrisflav assignee:chrisflav |
6-70197 6 days ago |
6-70197 6 days ago |
82-34290 82 days |
28389 |
euprunin author:euprunin |
chore(Algebra/Group/Subgroup): golf entire `subgroupOf_sup` |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
awaiting-author
label:t-algebra$ |
2/6 |
Mathlib/Algebra/Group/Subgroup/Ker.lean |
1 |
3 |
['Ruben-VandeVelde', 'chrisflav', 'euprunin', 'github-actions'] |
chrisflav assignee:chrisflav |
6-69742 6 days ago |
6-69742 6 days ago |
23-37322 23 days |
28305 |
euprunin author:euprunin |
chore(RingTheory/MvPolynomial): deprecate `weightedHomogeneousComponent_of_isWeightedHomogeneous_same` and golf entire `weightedHomogeneousComponent_of_isWeightedHomogeneous_ne` |
---
Show trace profiling of weightedHomogeneousComponent_of_isWeightedHomogeneous_same : 12 ms before, <10 ms after 🎉
### Trace profiling of `weightedHomogeneousComponent_of_isWeightedHomogeneous_same` before PR 28305
```diff
diff --git a/Mathlib/RingTheory/MvPolynomial/WeightedHomogeneous.lean b/Mathlib/RingTheory/MvPolynomial/WeightedHomogeneous.lean
index 6490df8bf8..1bdb4d75ae 100644
--- a/Mathlib/RingTheory/MvPolynomial/WeightedHomogeneous.lean
+++ b/Mathlib/RingTheory/MvPolynomial/WeightedHomogeneous.lean
@@ -434,2 +434,3 @@ theorem weightedHomogeneousComponent_of_mem [DecidableEq M] {m n : M}
+set_option trace.profiler true in
theorem weightedHomogeneousComponent_of_isWeightedHomogeneous_same
```
```
ℹ [1208/1208] Built Mathlib.RingTheory.MvPolynomial.WeightedHomogeneous
info: Mathlib/RingTheory/MvPolynomial/WeightedHomogeneous.lean:436:0: [Elab.async] [0.012999] elaborating proof of MvPolynomial.weightedHomogeneousComponent_of_isWeightedHomogeneous_same
[Elab.definition.value] [0.012383] MvPolynomial.weightedHomogeneousComponent_of_isWeightedHomogeneous_same
[Elab.step] [0.012139] classical
ext x
rw [coeff_weightedHomogeneousComponent]
by_cases zero_coeff : coeff x p = 0
· simp [zero_coeff]
· rw [hp zero_coeff, if_pos rfl]
[Elab.step] [0.012134] classical
ext x
rw [coeff_weightedHomogeneousComponent]
by_cases zero_coeff : coeff x p = 0
· simp [zero_coeff]
· rw [hp zero_coeff, if_pos rfl]
[Elab.step] [0.012128] classical
ext x
rw [coeff_weightedHomogeneousComponent]
by_cases zero_coeff : coeff x p = 0
· simp [zero_coeff]
· rw [hp zero_coeff, if_pos rfl]
[Elab.step] [0.012045]
ext x
rw [coeff_weightedHomogeneousComponent]
by_cases zero_coeff : coeff x p = 0
· simp [zero_coeff]
· rw [hp zero_coeff, if_pos rfl]
[Elab.step] [0.012034]
ext x
rw [coeff_weightedHomogeneousComponent]
by_cases zero_coeff : coeff x p = 0
· simp [zero_coeff]
· rw [hp zero_coeff, if_pos rfl]
Build completed successfully.
```
### Trace profiling of `weightedHomogeneousComponent_of_isWeightedHomogeneous_same` after PR 28305
```diff
diff --git a/Mathlib/RingTheory/MvPolynomial/WeightedHomogeneous.lean b/Mathlib/RingTheory/MvPolynomial/WeightedHomogeneous.lean
index 6490df8bf8..df101a703d 100644
--- a/Mathlib/RingTheory/MvPolynomial/WeightedHomogeneous.lean
+++ b/Mathlib/RingTheory/MvPolynomial/WeightedHomogeneous.lean
@@ -434,11 +434,7 @@ theorem weightedHomogeneousComponent_of_mem [DecidableEq M] {m n : M}
+set_option trace.profiler true in
theorem weightedHomogeneousComponent_of_isWeightedHomogeneous_same
{m : M} {p : MvPolynomial σ R} (hp : IsWeightedHomogeneous w p m) :
- weightedHomogeneousComponent w m p = p := by
- classical
- ext x
- rw [coeff_weightedHomogeneousComponent]
- by_cases zero_coeff : coeff x p = 0
- · simp [zero_coeff]
- · rw [hp zero_coeff, if_pos rfl]
+ weightedHomogeneousComponent w m p = p :=
+ IsWeightedHomogeneous.weightedHomogeneousComponent_same hp
@@ -446,9 +442,4 @@ theorem weightedHomogeneousComponent_of_isWeightedHomogeneous_ne
{m n : M} {p : MvPolynomial σ R} (hp : IsWeightedHomogeneous w p m) (hn : n ≠ m) :
- weightedHomogeneousComponent w n p = 0 := by
- classical
- ext x
- rw [coeff_weightedHomogeneousComponent]
- by_cases zero_coeff : coeff x p = 0
- · simp [zero_coeff]
- · rw [if_neg (by simp only [hp zero_coeff, hn.symm, not_false_eq_true]), coeff_zero]
+ weightedHomogeneousComponent w n p = 0 :=
+ IsWeightedHomogeneous.weightedHomogeneousComponent_ne n hp hn
```
```
✔ [1208/1208] Built Mathlib.RingTheory.MvPolynomial.WeightedHomogeneous
Build completed successfully.
```
---
Show trace profiling of weightedHomogeneousComponent_of_isWeightedHomogeneous_ne : 13 ms before, <10 ms after 🎉
### Trace profiling of `weightedHomogeneousComponent_of_isWeightedHomogeneous_ne` before PR 28305
```diff
diff --git a/Mathlib/RingTheory/MvPolynomial/WeightedHomogeneous.lean b/Mathlib/RingTheory/MvPolynomial/WeightedHomogeneous.lean
index 6490df8bf8..b83c5c6269 100644
--- a/Mathlib/RingTheory/MvPolynomial/WeightedHomogeneous.lean
+++ b/Mathlib/RingTheory/MvPolynomial/WeightedHomogeneous.lean
@@ -444,2 +444,3 @@ theorem weightedHomogeneousComponent_of_isWeightedHomogeneous_same
+set_option trace.profiler true in
theorem weightedHomogeneousComponent_of_isWeightedHomogeneous_ne
```
```
ℹ [1208/1208] Built Mathlib.RingTheory.MvPolynomial.WeightedHomogeneous
info: Mathlib/RingTheory/MvPolynomial/WeightedHomogeneous.lean:446:0: [Elab.async] [0.013611] elaborating proof of MvPolynomial.weightedHomogeneousComponent_of_isWeightedHomogeneous_ne
[Elab.definition.value] [0.012857] MvPolynomial.weightedHomogeneousComponent_of_isWeightedHomogeneous_ne
[Elab.step] [0.012517] classical
ext x
rw [coeff_weightedHomogeneousComponent]
by_cases zero_coeff : coeff x p = 0
· simp [zero_coeff]
· rw [if_neg (by simp only [hp zero_coeff, hn.symm, not_false_eq_true]), coeff_zero]
[Elab.step] [0.012512] classical
ext x
rw [coeff_weightedHomogeneousComponent]
by_cases zero_coeff : coeff x p = 0
· simp [zero_coeff]
· rw [if_neg (by simp only [hp zero_coeff, hn.symm, not_false_eq_true]), coeff_zero]
[Elab.step] [0.012508] classical
ext x
rw [coeff_weightedHomogeneousComponent]
by_cases zero_coeff : coeff x p = 0
· simp [zero_coeff]
· rw [if_neg (by simp only [hp zero_coeff, hn.symm, not_false_eq_true]), coeff_zero]
[Elab.step] [0.012450]
ext x
rw [coeff_weightedHomogeneousComponent]
by_cases zero_coeff : coeff x p = 0
· simp [zero_coeff]
· rw [if_neg (by simp only [hp zero_coeff, hn.symm, not_false_eq_true]), coeff_zero]
[Elab.step] [0.012443]
ext x
rw [coeff_weightedHomogeneousComponent]
by_cases zero_coeff : coeff x p = 0
· simp [zero_coeff]
· rw [if_neg (by simp only [hp zero_coeff, hn.symm, not_false_eq_true]), coeff_zero]
Build completed successfully.
```
### Trace profiling of `weightedHomogeneousComponent_of_isWeightedHomogeneous_ne` after PR 28305
```diff
diff --git a/Mathlib/RingTheory/MvPolynomial/WeightedHomogeneous.lean b/Mathlib/RingTheory/MvPolynomial/WeightedHomogeneous.lean
index 6490df8bf8..066f4824e9 100644
--- a/Mathlib/RingTheory/MvPolynomial/WeightedHomogeneous.lean
+++ b/Mathlib/RingTheory/MvPolynomial/WeightedHomogeneous.lean
@@ -436,19 +436,10 @@ theorem weightedHomogeneousComponent_of_isWeightedHomogeneous_same
{m : M} {p : MvPolynomial σ R} (hp : IsWeightedHomogeneous w p m) :
- weightedHomogeneousComponent w m p = p := by
- classical
- ext x
- rw [coeff_weightedHomogeneousComponent]
- by_cases zero_coeff : coeff x p = 0
- · simp [zero_coeff]
- · rw [hp zero_coeff, if_pos rfl]
+ weightedHomogeneousComponent w m p = p :=
+ IsWeightedHomogeneous.weightedHomogeneousComponent_same hp
+set_option trace.profiler true in
theorem weightedHomogeneousComponent_of_isWeightedHomogeneous_ne
{m n : M} {p : MvPolynomial σ R} (hp : IsWeightedHomogeneous w p m) (hn : n ≠ m) :
- weightedHomogeneousComponent w n p = 0 := by
- classical
- ext x
- rw [coeff_weightedHomogeneousComponent]
- by_cases zero_coeff : coeff x p = 0
- · simp [zero_coeff]
- · rw [if_neg (by simp only [hp zero_coeff, hn.symm, not_false_eq_true]), coeff_zero]
+ weightedHomogeneousComponent w n p = 0 :=
+ IsWeightedHomogeneous.weightedHomogeneousComponent_ne n hp hn
```
```
✔ [1208/1208] Built Mathlib.RingTheory.MvPolynomial.WeightedHomogeneous
Build completed successfully.
```
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
awaiting-author
|
6/17 |
Mathlib/RingTheory/MvPolynomial/WeightedHomogeneous.lean |
1 |
4 |
['chrisflav', 'github-actions', 'mattrobball'] |
chrisflav assignee:chrisflav |
6-69542 6 days ago |
6-69542 6 days ago |
24-72362 24 days |
28140 |
YaelDillies author:YaelDillies |
feat: a `PointedCone`-valued version of `Submodule.span` |
This is merely to guide typing.
From Toric
---
[](https://gitpod.io/from-referrer/)
|
t-convex-geometry
toric
|
11/2 |
Mathlib/Geometry/Convex/Cone/Dual.lean,Mathlib/Geometry/Convex/Cone/Pointed.lean |
2 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
6-67450 6 days ago |
6-67481 6 days ago |
34-62373 34 days |
28295 |
artie2000 author:artie2000 |
feat(Algebra/Order/Ring/Ordering): basic results about ring (pre)orderings |
* Basic automation for membership of ring orderings
* Alternative constructors for ring preorderings and ring orderings
* Basic results about ring preorderings and their supports, including the special case over a field
---
[](https://gitpod.io/from-referrer/)
- [x] depends on: #27282 |
t-algebra
awaiting-author
label:t-algebra$ |
216/0 |
Mathlib.lean,Mathlib/Algebra/Group/Subgroup/Defs.lean,Mathlib/Algebra/Module/Submodule/Lattice.lean,Mathlib/Algebra/Order/Ring/Ordering/Basic.lean |
4 |
49 |
['Rob23oba', 'YaelDillies', 'artie2000', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'vihdzp'] |
nobody |
6-66496 6 days ago |
13-38222 13 days ago |
4-49774 4 days |
28970 |
Whysoserioushah author:Whysoserioushah |
feat(Algebra/Algebra/ReducedNorm) : Defines reduced norm and trace |
TODO :
1. add the theorem proving reduced charpoly is independent from the choice of AlgEquiv (blocked by this [discussion](https://leanprover.zulipchat.com/#narrow/channel/217875-Is-there-code-for-X.3F/topic/Algebra.2ETensorProduct.2Eassoc/with/536349758))
2. prove reduced charpoly is "actually" in the polynomial ring of base field (blocked by this [discussion](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/.E2.9C.94.20Refactor.20Subfield))
therefore content about this topic is basically the best I could do for now :-(
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
66/0 |
Mathlib.lean,Mathlib/Algebra/Algebra/ReducedNorm.lean |
2 |
15 |
['Whysoserioushah', 'chrisflav', 'eric-wieser', 'github-actions', 'kbuzzard'] |
chrisflav assignee:chrisflav |
6-66266 6 days ago |
6-67614 6 days ago |
17-68994 17 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$ |
269/4 |
Mathlib.lean,Mathlib/Analysis/NormedSpace/PiTensorProduct/ProjectiveSeminorm.lean,Mathlib/Data/SubtypeNeLift.lean,Mathlib/LinearAlgebra/PiTensorProduct/Basic.lean,Mathlib/LinearAlgebra/PiTensorProduct/Finite.lean,Mathlib/LinearAlgebra/PiTensorProduct/Generators.lean,Mathlib/LinearAlgebra/TensorPower/Basic.lean,Mathlib/RingTheory/PiTensorProduct.lean,Mathlib/SetTheory/Cardinal/Finite.lean |
9 |
19 |
['eric-wieser', 'github-actions', 'joelriou', 'leanprover-community-bot-assistant', 'mathlib4-merge-conflict-bot'] |
mattrobball assignee:mattrobball |
6-34912 6 days ago |
13-84885 13 days ago |
63-27856 63 days |
26923 |
oliver-butterley author:oliver-butterley |
feat(Dynamics/BirkhoffSum): add the pointwise ergodic theorem (Birkhoff's) |
The Pointwise Ergodic Theorem, also known as Birkhoff's Ergodic Theorem.
Co-authored-by: Lua Viana Reis
- [x] depends on: #26074
- [x] depends on: #26807
- [x] depends on: #26810
- [x] depends on: #26840
- [x] depends on: #26842
- [x] depends on: #26848
- [x] depends on: #26851
- [x] depends on: #26852
- [x] depends on: #26853
- [x] depends on: #27008
- [x] depends on: #28901
Zulip: [PR thread](https://leanprover.zulipchat.com/#narrow/channel/144837-PR-reviews/topic/.2326923.20The.20pointwise.20ergodic.20theorem.20.28Birkhoff's.29/with/527835158)
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-dynamics
|
401/0 |
Mathlib.lean,Mathlib/Dynamics/BirkhoffSum/Pointwise.lean |
2 |
7 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
urkud assignee:urkud |
6-34911 6 days ago |
18-21265 18 days ago |
24-77138 24 days |
28339 |
JovanGerb author:JovanGerb |
feat(gcongr): support `@[gcongr]` for `Monotone` and friends |
This PR adds the feature to `gcongr` that you can now tag lemmas whose conclusion is `Monotone f`, `Antitone f`, etc.
---
[](https://gitpod.io/from-referrer/)
|
t-meta |
119/88 |
Mathlib/Algebra/Order/Floor/Ring.lean,Mathlib/Algebra/Order/Floor/Semiring.lean,Mathlib/Algebra/Order/Module/Algebra.lean,Mathlib/Algebra/Order/Ring/Cast.lean,Mathlib/Algebra/Ring/Subring/Basic.lean,Mathlib/Analysis/Complex/Exponential.lean,Mathlib/Analysis/SpecialFunctions/Log/ERealExp.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Arctan.lean,Mathlib/Data/Finsupp/Order.lean,Mathlib/Data/Multiset/Defs.lean,Mathlib/Data/Nat/Cast/Order/Basic.lean,Mathlib/Data/Rat/Cast/Order.lean,Mathlib/Data/Real/Sqrt.lean,Mathlib/LinearAlgebra/Basis/Flag.lean,Mathlib/MeasureTheory/Function/SimpleFunc.lean,Mathlib/Order/Filter/Map.lean,Mathlib/Order/Hom/Basic.lean,Mathlib/Order/KrullDimension.lean,Mathlib/Tactic/GCongr/Core.lean,MathlibTest/GCongr/inequalities.lean |
20 |
4 |
['github-actions', 'kckennylau', 'mathlib4-merge-conflict-bot'] |
adamtopaz assignee:adamtopaz |
6-34910 6 days ago |
17-69540 17 days ago |
30-39760 30 days |
28876 |
ScottCarnahan author:ScottCarnahan |
feat (Algebra/Group/Action/Basic): add IsLeftCancelSMul |
This PR adds classes `IsLeftCancelSMul` and `IsLeftCancelVAdd`, for actions that are injective on the left. This property automatically holds for group actions, and for the left multiplication action of a left cancellative monoid.
---
[](https://gitpod.io/from-referrer/)
|
|
41/15 |
Mathlib/Algebra/Group/Action/Defs.lean,Mathlib/Algebra/Order/AddTorsor.lean,Mathlib/Data/Finset/SMulAntidiagonal.lean,Mathlib/Data/Set/SMulAntidiagonal.lean,Mathlib/RingTheory/HahnSeries/Multiplication.lean |
5 |
1 |
['github-actions'] |
dagurtomas assignee:dagurtomas |
6-34908 6 days ago |
14-4175 14 days ago |
19-49638 19 days |
28833 |
yury-harmonic author:yury-harmonic |
feat(MvPolynomial/Expand): more lemmas |
---
- [x] depends on: #28832
- [x] depends on: #28830
[](https://gitpod.io/from-referrer/)
|
|
88/18 |
Mathlib/Algebra/MvPolynomial/Eval.lean,Mathlib/Algebra/MvPolynomial/Expand.lean |
2 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
dwrensha assignee:dwrensha |
6-34908 6 days ago |
19-51649 19 days ago |
19-53402 19 days |
29103 |
grunweg author:grunweg |
chore: tests for casting and the field_simp discharger |
Add further tests for the `field_simps` discharger and casting, inspired by #6034.
Golf a few field_simp proofs further, such as by using `norm_cast` as discharger.
In particular, this PR includes all mathlib changes from #6034.
Golf two proofs that we noticed in passing.
---
[](https://gitpod.io/from-referrer/)
|
t-meta |
25/14 |
Mathlib/Analysis/Analytic/Composition.lean,Mathlib/Analysis/Fourier/AddCircle.lean,Mathlib/Analysis/InnerProductSpace/Dual.lean,Mathlib/Analysis/SpecialFunctions/Stirling.lean,Mathlib/Analysis/SpecificLimits/RCLike.lean,Mathlib/NumberTheory/PythagoreanTriples.lean,Mathlib/RingTheory/RootsOfUnity/Complex.lean,MathlibTest/FieldSimp.lean |
8 |
3 |
['github-actions', 'grunweg', 'hrmacbeth'] |
adamtopaz assignee:adamtopaz |
6-34906 6 days ago |
14-78847 14 days ago |
15-1131 15 days |
29122 |
yonggyuchoimath author:yonggyuchoimath |
feat(CategoryTheory/MorphismProperty/Representable): add relative representability of diagonal map |
Adds a criterion for the diagonal morphism `X ⟶ X × X` to be relatively representable with respect to a functor `F : C ⥤ D` under mild assumptions.
`CategoryTheory.Functor.relativelyRepresentable.diag_iff` proves that when:
- `C` has pullbacks and binary products
- `D` has pullbacks, binary products and a terminal object
- `F : C ⥤ D` is full and preserves pullbacks and binary products
the diagonal morphism `X ⟶ X × X` is relatively representable if and only if every morphism of the form `F.obj a ⟶ X` is relatively representable. |
new-contributor
t-category-theory
|
67/0 |
Mathlib/CategoryTheory/MorphismProperty/Representable.lean |
1 |
1 |
['github-actions'] |
riccardobrasca assignee:riccardobrasca |
6-34905 6 days ago |
14-24675 14 days ago |
14-24711 14 days |
29121 |
Ruben-VandeVelde author:Ruben-VandeVelde |
feat: MvPolynomial.symmetricSubalgebra.{aevalMultiset,sumPolynomial} |
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory |
192/0 |
Mathlib.lean,Mathlib/RingTheory/MvPolynomial/Symmetric/Eval.lean |
2 |
1 |
['github-actions'] |
chrisflav assignee:chrisflav |
6-34905 6 days ago |
14-34577 14 days ago |
14-34615 14 days |
29369 |
vlad902 author:vlad902 |
feat(SimpleGraph): `IsSubwalk` of common Walk decompositions |
Add some helper lemmas to show that decompositions of walks are sub-walks. |
t-combinatorics |
61/17 |
Mathlib/Combinatorics/SimpleGraph/Connectivity/WalkDecomp.lean,Mathlib/Combinatorics/SimpleGraph/Walk.lean |
2 |
1 |
['github-actions'] |
nobody |
6-16294 6 days ago |
7-60389 7 days ago |
7-60437 7 days |
29376 |
vlad902 author:vlad902 |
feat(SimpleGraph): Helper lemmas for `Walk.IsSubwalk` |
|
t-combinatorics |
29/0 |
Mathlib/Combinatorics/SimpleGraph/Walk.lean |
1 |
1 |
['github-actions'] |
nobody |
6-16123 6 days ago |
7-12611 7 days ago |
7-12650 7 days |
26836 |
mans0954 author:mans0954 |
feat(Order/Lattice): conditions for an equivalence relation to be a lattice congruence |
Define a structure asserting that a binary relation is a lattice congruence and provide sufficient and necessary conditions.
An application is given in #26983
---
- [x] depends on: #27219
[](https://gitpod.io/from-referrer/)
|
t-order
awaiting-author
|
133/0 |
Mathlib.lean,Mathlib/Order/Lattice/Congruence.lean,docs/references.bib |
3 |
50 |
['YaelDillies', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'mans0954', 'mathlib4-dependent-issues-bot'] |
nobody |
6-14866 6 days ago |
46-8853 1 month ago |
19-42188 19 days |
29306 |
YaelDillies author:YaelDillies |
chore(GroupTheory/GroupAction/Basic): don't import `Module` |
This is useful to be able to replace `NoZeroSMulDivisors` with `Module.IsTorsionFree` later.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
16/17 |
Mathlib/GroupTheory/GroupAction/Basic.lean,Mathlib/LinearAlgebra/Projectivization/Cardinality.lean |
2 |
7 |
['YaelDillies', 'eric-wieser', 'github-actions'] |
eric-wieser assignee:eric-wieser |
6-12019 6 days ago |
6-12097 6 days ago |
9-59845 9 days |
29212 |
Whysoserioushah author:Whysoserioushah |
feat(Algebra/CrossProductAlgebra/Defs) : Define Cross Product Algebra |
PS: All to-dos listed in the file has been fully sorry-freed and will be (slowly) upstreamed by either me or Yaël
Co-authored-by: Yaël Dillies
Co-authored-by: Jujian Zhang
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
awaiting-author
label:t-algebra$ |
270/0 |
Mathlib.lean,Mathlib/RepresentationTheory/CrossProductAlgebra/Defs.lean,docs/references.bib |
3 |
8 |
['Whysoserioushah', 'YaelDillies', 'eric-wieser', 'github-actions'] |
nobody |
6-9418 6 days ago |
6-9418 6 days ago |
5-63264 5 days |
29397 |
vihdzp author:vihdzp |
chore(Algebra/Polynomial/Basic): make some arguments implicit |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
8/8 |
Mathlib/Algebra/Polynomial/Basic.lean,Mathlib/Algebra/Polynomial/Lifts.lean,Mathlib/RingTheory/Polynomial/Basic.lean,Mathlib/RingTheory/Polynomial/ContentIdeal.lean |
4 |
1 |
['github-actions'] |
nobody |
6-2623 6 days ago |
6-4892 6 days ago |
6-4928 6 days |
29347 |
themathqueen author:themathqueen |
refactor(Algebra/Star/StarAlgHom): let `StarAlgEquiv` extend `StarRingEquiv` instead of `RingEquiv` |
Instead of having `StarAlgEquiv` extend `RingEquiv` and have properties `map_star'` and `map_smul'`, it now extends `StarRingEquiv` with only `map_smul'`.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
29/36 |
Mathlib/Algebra/Star/StarAlgHom.lean,Mathlib/Analysis/CStarAlgebra/CStarMatrix.lean |
2 |
4 |
['github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot'] |
nobody |
6-1370 6 days ago |
6-47832 6 days ago |
8-70791 8 days |
28511 |
YaelDillies author:YaelDillies |
feat(Finsupp): `congr!`-compatible version of `prod_congr` |
`congr!` doesn't like the `g1 x (f x)` appearing in the hypothesis of `Finsupp.prod_congr`: `f x` isn't a free variable.
Note: A few proofs broke due to `simp` using `congr` lemmas internally.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
17/11 |
Mathlib/Algebra/BigOperators/Finsupp/Basic.lean,Mathlib/Algebra/Category/MonCat/Adjunctions.lean,Mathlib/Data/Finsupp/Multiset.lean,Mathlib/Data/Nat/Choose/Multinomial.lean,Mathlib/RepresentationTheory/Homological/GroupHomology/LowDegree.lean |
5 |
12 |
['JovanGerb', 'YaelDillies', 'eric-wieser', 'github-actions', 'kmill'] |
kmill assignee:kmill |
5-86003 5 days ago |
28-6058 28 days ago |
28-6096 28 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
|
166/5 |
Mathlib/SetTheory/ZFC/Basic.lean,Mathlib/SetTheory/ZFC/Ordinal.lean,Mathlib/SetTheory/ZFC/PSet.lean,Mathlib/SetTheory/ZFC/Rank.lean |
4 |
23 |
['alreadydone', 'github-actions', 'leanprover-community-bot-assistant', 'staroperator', 'vihdzp'] |
nobody |
5-76743 5 days ago |
6-3455 6 days ago |
32-67217 32 days |
28728 |
or4nge19 author:or4nge19 |
feat(PerronFrobenius): introduce StronglyConnected Quiver and Irreducible and Primitive Matrices and their basic properties and relations |
This PR develops a graph-theoretic interface for studying nonnegative square matrices over `ℝ`
through the quiver formed by their strictly positive entries. It shows the equivalence
between positivity of suitable matrix powers and existence of directed paths in this quiver.
------------
- [ ] depends on: #28696
[](https://gitpod.io/from-referrer/)
|
file-removed
new-contributor
awaiting-author
|
305/256 |
Mathlib.lean,Mathlib/Combinatorics/Quiver/Path/StronglyConnected.lean,Mathlib/Combinatorics/Quiver/Path/Vertices.lean,Mathlib/Data/List/Basic.lean,Mathlib/LinearAlgebra/Matrix/Irreducible/Defs.lean |
5 |
5 |
['github-actions', 'j-loreaux', 'mathlib4-dependent-issues-bot', 'or4nge19'] |
nobody |
5-76006 5 days ago |
5-76006 5 days ago |
0-32474 9 hours |
29362 |
stepanholub author:stepanholub |
Periods of lists and the Periodicity Lemma |
Period of a word (List) is defined and a proof of the Periodicity Lemma (aka Fine-Wilf Theorem) is provided. Fine-Wilf is the basic fact about a word having two periods.
---
|
t-data
new-contributor
|
223/0 |
Mathlib.lean,Mathlib/Data/List/PeriodicityLemma.lean |
2 |
99 |
['Timeroot', 'github-actions', 'madvorak', 'plp127', 'stepanholub'] |
nobody |
5-70652 5 days ago |
8-4423 8 days ago |
8-4465 8 days |
29228 |
Timeroot author:Timeroot |
feat(Logic/Basic): HEq iff Exists a cast |
Proves that `a ≍ b ↔ ∃ (h : β = α), a = cast h b`. This is pretty similar to existing e.g. `heq_of_eq_cast (e : β = α) : a = cast e b → a ≍ b`, but this is more amenable to rewriting with simp (e.g. under binders).
---
[](https://gitpod.io/from-referrer/)
|
t-logic |
9/0 |
Mathlib/Logic/Basic.lean |
1 |
3 |
['Timeroot', 'github-actions', 'plp127'] |
nobody |
5-68039 5 days ago |
11-30117 11 days ago |
11-30154 11 days |
27073 |
pechersky author:pechersky |
feat(Archive/Examples/Local): files showcasing properties of local fields |
for p-adics, completions of number fields, laurent series, and fraction rings of witt vectors
Should get filled in as more data/instances are declared
---
[](https://gitpod.io/from-referrer/)
|
t-number-theory |
139/0 |
Archive.lean,Archive/Examples/Local/Laurent.lean,Archive/Examples/Local/NumberField.lean,Archive/Examples/Local/Padic.lean,Archive/Examples/Local/Witt.lean |
5 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
alexjbest assignee:alexjbest |
5-60876 5 days ago |
5-60903 5 days ago |
56-77671 56 days |
29407 |
pechersky author:pechersky |
feat(RingTheory): hom from local ring to ZMod is a local hom |
complex imports make it difficult to find a good file to place in
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory |
5/0 |
Mathlib/RingTheory/LocalRing/Module.lean |
1 |
1 |
['github-actions'] |
nobody |
5-57910 5 days ago |
5-57973 5 days ago |
5-57960 5 days |
29410 |
jsm28 author:jsm28 |
feat(Data/Nat/Init): `n.AtLeastTwo` implies `NeZero (n - 1)` |
Add an instance for `NeZero (n - 1)` deduced from `n.AtLeastTwo`.
---
[](https://gitpod.io/from-referrer/)
|
t-data |
2/0 |
Mathlib/Data/Nat/Init.lean |
1 |
1 |
['github-actions'] |
nobody |
5-49367 5 days ago |
5-49431 5 days ago |
5-49412 5 days |
29404 |
pechersky author:pechersky |
feat(Data/Nat): p.Coprime factorial and choose |
And descFactorial, for n < p
---
[](https://gitpod.io/from-referrer/)
|
t-data
maintainer-merge
t-algebra
easy
label:t-algebra$ |
16/0 |
Mathlib/Data/Nat/Choose/Dvd.lean,Mathlib/Data/Nat/Prime/Factorial.lean |
2 |
2 |
['Ruben-VandeVelde', 'github-actions'] |
nobody |
5-45565 5 days ago |
5-45565 5 days ago |
5-59140 5 days |
29225 |
euprunin author:euprunin |
chore: remove redundant `cases` invocations |
---
**Note:** Although technically redundant, some of these may be worth keeping for readability, or other reasons. Let me know if you think any should stay.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
2/16 |
Mathlib/Algebra/CharP/Lemmas.lean,Mathlib/Algebra/Lie/Subalgebra.lean,Mathlib/Algebra/Module/Submodule/Equiv.lean,Mathlib/Algebra/MonoidAlgebra/Degree.lean,Mathlib/Algebra/Polynomial/Basic.lean |
5 |
4 |
['github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot'] |
nobody |
5-43130 5 days ago |
5-43130 5 days ago |
11-53072 11 days |
28834 |
euprunin author:euprunin |
chore(Data/Finset): golf 10 lines from `powerset_insert` using `grind` |
---
[](https://gitpod.io/from-referrer/)
|
t-data |
1/11 |
Mathlib/Data/Finset/Powerset.lean |
1 |
4 |
['github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot'] |
nobody |
5-41614 5 days ago |
5-41614 5 days ago |
20-19739 20 days |
28835 |
euprunin author:euprunin |
chore(Data/List): golf 13 lines from `bidirectionalRec_cons_append` using `grind` |
---
[](https://gitpod.io/from-referrer/)
|
t-data |
1/14 |
Mathlib/Data/List/Induction.lean |
1 |
4 |
['github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot'] |
nobody |
5-40115 5 days ago |
5-40115 5 days ago |
20-19593 20 days |
28841 |
euprunin author:euprunin |
chore(Data/List): golf entire `mem_getLast?_append_of_mem_getLast` and `mem_head?_append_of_mem_head?` using `grind` |
---
[](https://gitpod.io/from-referrer/)
|
t-data |
2/7 |
Mathlib/Data/List/Basic.lean |
1 |
6 |
['github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot'] |
nobody |
5-38609 5 days ago |
5-38609 5 days ago |
20-7363 20 days |
29409 |
Julian author:Julian |
feat(Mathlib/Analysis): deriv_eq_self and deriv_exp_iff |
---
[](https://gitpod.io/from-referrer/)
|
t-analysis |
32/0 |
Mathlib/Analysis/SpecialFunctions/ExpDeriv.lean |
1 |
2 |
['eric-wieser', 'github-actions'] |
nobody |
5-37539 5 days ago |
5-50119 5 days ago |
5-50163 5 days |
28219 |
joelriou author:joelriou |
feat(CategoryTheory): monomorphisms in Type are stable under transfinite compositions |
---
- [x] depends on: #26030
[](https://gitpod.io/from-referrer/)
|
t-category-theory |
71/0 |
Mathlib.lean,Mathlib/CategoryTheory/Limits/Types/Shapes.lean,Mathlib/CategoryTheory/Types/Monomorphisms.lean |
3 |
5 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
TwoFX assignee:TwoFX |
5-34914 5 days ago |
14-45366 14 days ago |
14-62210 14 days |
29166 |
YaelDillies author:YaelDillies |
feat: group objects form a cartesian-monoidal category |
From Toric
---
[](https://gitpod.io/from-referrer/)
|
toric
t-category-theory
|
71/0 |
Mathlib/CategoryTheory/Monoidal/Grp_.lean |
1 |
1 |
['github-actions'] |
kim-em assignee:kim-em |
5-34908 5 days ago |
12-86102 12 days ago |
12-86085 12 days |
29185 |
eric-wieser author:eric-wieser |
feat: add missing `norm_cast` on subobject coercion lemmas to set |
This is not exhaustive, but performed manually with some regex searches.
Only one proof breaks, and only because `convert` goes further than it previously did.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
56/52 |
Mathlib/Algebra/Algebra/NonUnitalSubalgebra.lean,Mathlib/Algebra/Algebra/Subalgebra/Lattice.lean,Mathlib/Algebra/Algebra/Subalgebra/Pointwise.lean,Mathlib/Algebra/Algebra/Subalgebra/Prod.lean,Mathlib/Algebra/Field/Subfield/Basic.lean,Mathlib/Algebra/Field/Subfield/Defs.lean,Mathlib/Algebra/Group/Subgroup/Basic.lean,Mathlib/Algebra/Group/Subgroup/Lattice.lean,Mathlib/Algebra/Group/Subgroup/Pointwise.lean,Mathlib/Algebra/Group/Submonoid/Defs.lean,Mathlib/Algebra/Group/Submonoid/Operations.lean,Mathlib/Algebra/Group/Submonoid/Pointwise.lean,Mathlib/Algebra/Group/Subsemigroup/Defs.lean,Mathlib/Algebra/Group/Subsemigroup/Operations.lean,Mathlib/Algebra/GroupWithZero/Subgroup.lean,Mathlib/Algebra/GroupWithZero/Submonoid/Pointwise.lean,Mathlib/Algebra/Lie/Submodule.lean,Mathlib/Algebra/Module/Submodule/Pointwise.lean,Mathlib/Algebra/Ring/Subring/Basic.lean,Mathlib/Algebra/Ring/Subring/Pointwise.lean,Mathlib/Algebra/Ring/Subsemiring/Basic.lean,Mathlib/Algebra/Ring/Subsemiring/Defs.lean,Mathlib/Algebra/Ring/Subsemiring/Pointwise.lean,Mathlib/Algebra/Star/NonUnitalSubalgebra.lean,Mathlib/Algebra/Star/NonUnitalSubsemiring.lean,Mathlib/Algebra/Star/Subalgebra.lean,Mathlib/Algebra/Star/Subsemiring.lean,Mathlib/Topology/Algebra/Group/ClosedSubgroup.lean |
28 |
1 |
['github-actions'] |
dagurtomas assignee:dagurtomas |
5-34907 5 days ago |
12-57614 12 days ago |
12-57596 12 days |
24669 |
qawbecrdtey author:qawbecrdtey |
feat(Analysis/Normed/Operator/LinearIsometry): added definition `LinearIsometryEquiv.prodComm` |
---
[](https://gitpod.io/from-referrer/)
This commit defines a `LinearIsometryEquiv`, and states some trivial theorems about it.
```lean
def prodComm [Module R E₂] : E × E₂ ≃ₗᵢ[R] E₂ × E
```
|
maintainer-merge
t-analysis
awaiting-author
|
8/1 |
Mathlib/Analysis/Normed/Operator/LinearIsometry.lean |
1 |
12 |
['Ruben-VandeVelde', 'eric-wieser', 'faenuccio', 'github-actions', 'j-loreaux', 'jcommelin', 'qawbecrdtey'] |
faenuccio assignee:faenuccio |
5-32953 5 days ago |
95-20785 3 months ago |
32-83569 32 days |
27742 |
ChrisHughes24 author:ChrisHughes24 |
feat(Nat/nth): inequalities about Nat.nth |
---
[](https://gitpod.io/from-referrer/)
|
t-data |
51/0 |
Mathlib/Data/Nat/Nth.lean |
1 |
3 |
['ChrisHughes24', 'github-actions'] |
nobody |
5-11661 5 days ago |
43-85327 1 month ago |
43-85370 43 days |
29422 |
jsm28 author:jsm28 |
fix(Data/Finset/Max): Use `DecidableEq` for `insert` lemmas |
These `insert` in these lemma statements uses a `DecidableEq` instance derived from `LinearOrder`; make them syntactically more general by passing in a `DecidableEq` instance separately. (Some `insert` lemmas in this file already take `DecidableEq` hypotheses.)
---
[](https://gitpod.io/from-referrer/)
|
t-data |
4/4 |
Mathlib/Data/Finset/Max.lean |
1 |
2 |
['eric-wieser', 'github-actions'] |
nobody |
5-4868 5 days ago |
5-32866 5 days ago |
5-32848 5 days |
29352 |
fpvandoorn author:fpvandoorn |
refactor: simplify dictionary in fixAbbreviation |
* Improve capitalization algorithm: you now don't have to give entries twice in `fixAbbreviation` (now `abbreviationDict`).
* The new algorithm uses the fact that we can easily find the `lowerCamelCase` name from the `UpperCamelCase` name, namely by applying `String.decapitalizeSeq`. This means that both `nameDict` and `abbreviationDict` have as input `lowerCamelCase` and as output `UpperCamelCase`.
* This removes the need to especially fix `NSMul`/`ZSMul` and similar.
* `abbreviationDict` still needs two entries if both `snake_case` and either `camelCase` need to be translated.
---
[](https://gitpod.io/from-referrer/)
|
t-meta |
146/160 |
Mathlib/Tactic/ToAdditive/GuessName.lean,MathlibTest/toAdditive.lean |
2 |
17 |
['JovanGerb', 'fpvandoorn', 'github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot'] |
nobody |
5-1936 5 days ago |
6-38878 6 days ago |
1-31909 1 day |
26757 |
fweth author:fweth |
feat(CategoryTheory/Topos): define elementary topos |
This commit begins the formalization of the notion of an *elementary topos*, following the definition in \[Mac Lane & Moerdijk, *Sheaves in Geometry and Logic* (1992), Ch. IV, Section 1]. It introduces the file `Mathlib/CategoryTheory/Topos/Basic.lean`, which currently includes:
* The definition of an elementary topos.
* Proof that the power object map is a functor
* Theorem about pullbacks of characterstic maps
Subobject classifiers, which are used in the definition, have already been defined in `CategoryTheory/Topos/Classifier.lean`
Work in progress: further formalization of the section is planned.
Questions:
* Should the definition of power objects be separated into its own file/module, perhaps under `CategoryTheory/Topos/PowerObject.lean`?
* Is the notation `P` / `P_morph` / `P_functor` for the power object functor on objects / morphisms / total acceptable?
* Should the comments and docstrings rather use the notation from the book, where `g ∘ f` denotes arrow composition from righ to left, or the Lean variant `f ≫ g`?
Klaus Gy klausgy@gmail.com
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-category-theory
|
391/68 |
Mathlib.lean,Mathlib/CategoryTheory/Closed/PowerObjects.lean,Mathlib/CategoryTheory/Limits/Shapes/BinaryProducts.lean,Mathlib/CategoryTheory/Limits/Shapes/Equalizers.lean,Mathlib/CategoryTheory/Limits/Shapes/Pullback/CommSq.lean,Mathlib/CategoryTheory/Limits/Shapes/Pullback/Equalizer.lean,Mathlib/CategoryTheory/Monoidal/Cartesian/Basic.lean,Mathlib/CategoryTheory/Subobject/Basic.lean,Mathlib/CategoryTheory/Topos/Classifier.lean |
9 |
13 |
['fweth', 'github-actions', 'joelriou', 'leanprover-community-bot-assistant', 'mathlib4-merge-conflict-bot'] |
nobody |
4-82113 4 days ago |
5-72087 5 days ago |
25-44253 25 days |
29427 |
kim-em author:kim-em |
feat: grind annotations for `Finset.sdiff` |
|
t-data |
29/27 |
Mathlib/CategoryTheory/Limits/Bicones.lean,Mathlib/Combinatorics/SetFamily/Compression/UV.lean,Mathlib/Data/Finset/Card.lean,Mathlib/Data/Finset/Empty.lean,Mathlib/Data/Finset/Fold.lean,Mathlib/Data/Finset/Image.lean,Mathlib/Data/Finset/Insert.lean,Mathlib/Data/Finset/Lattice/Basic.lean,Mathlib/Data/Finset/SDiff.lean,scripts/noshake.json |
10 |
1 |
['github-actions'] |
nobody |
4-81743 4 days ago |
5-20271 5 days ago |
5-20310 5 days |
29400 |
ShreckYe author:ShreckYe |
feat(`Algebra/BigOperators`): products of the results of insertion and removal on tuples and lists, and some needed lemmas |
|
large-import |
102/0 |
Mathlib.lean,Mathlib/Algebra/BigOperators/Fin.lean,Mathlib/Algebra/BigOperators/Group/List/Basic.lean,Mathlib/Algebra/BigOperators/Group/List/Defs.lean,Mathlib/Algebra/BigOperators/Group/Vector/Basic.lean,Mathlib/Data/Fin/Tuple/Basic.lean |
6 |
5 |
['ShreckYe', 'eric-wieser', 'github-actions'] |
nobody |
4-79309 4 days ago |
5-82701 5 days ago |
5-82749 5 days |
27390 |
alreadydone author:alreadydone |
feat(FieldTheory/Galois): normal basis theorem |
Co-authored-by: Madison Crim @maddycrim
Co-authored-by: Aaron Liu @plp127
Co-authored-by: Justus Springer @justus-springer
from [*Formalizing Class Field Theory*](https://www.claymath.org/events/formalizing-class-field-theory/)
---
- [x] depends on: #27355
- [x] depends on: #27368
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
156/1 |
Mathlib.lean,Mathlib/Algebra/Module/PID.lean,Mathlib/Algebra/Polynomial/Module/AEval.lean,Mathlib/FieldTheory/Galois/NormalBasis.lean,Mathlib/LinearAlgebra/Dual/Lemmas.lean,Mathlib/LinearAlgebra/LinearIndependent/Basic.lean,docs/references.bib |
7 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
dagurtomas assignee:dagurtomas |
4-78505 4 days ago |
4-78569 4 days ago |
30-38535 30 days |
29373 |
staroperator author:staroperator |
doc(ModelTheory): clarify free and (in-scope) bound variables in `BoundedFormula` |
The current design of `BoundedFormula` is actually a locally nameless representation. Following PL convention, we should call the `α` indexed variables as free variables, and the `Fin n` indexed variables as (in-scope) bound variables.
Also clarify that the bound variables are actually de Bruijn levels.
Some references:
-
- [Locally nameless in CSLib](https://github.com/leanprover/cslib/blob/4734d98a80d82e8bb15cbb64b6cfaa30c08691a8/Cslib/Languages/LambdaCalculus/LocallyNameless/Untyped/Basic.lean)
- [Locally nameless in Lean core](https://github.com/leanprover/lean4/blob/540e9e85f3317d04133aa2a69d5a24fb31e92d8b/src/Lean/Expr.lean#L238)
---
[](https://gitpod.io/from-referrer/)
|
t-logic
documentation
|
32/31 |
Mathlib/ModelTheory/Semantics.lean,Mathlib/ModelTheory/Syntax.lean |
2 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
4-76639 4 days ago |
4-76659 4 days ago |
7-29251 7 days |
28289 |
robin-carlier author:robin-carlier |
chore(CategoryTheory/Bicategory/Functor/Strict): generalize some results to op/lax functors |
We generalize some of the results in `CategoryTheory/Bicategory/Functor/Strict/` to op/lax functors.
The results for lax functors will be useful when studying types of strictly unitary lay functors from `LocallyDiscrete (Fin (n + 1))` to a bicategory `B`, i.e the type of lax-composable arrows in `B`.
This PR is part of an ongoing effort to formalize the Duskin nerve of a bicategory.
---
- [ ] depends on: #28287
[](https://gitpod.io/from-referrer/)
|
large-import
t-category-theory
delegated
|
148/13 |
Mathlib/CategoryTheory/Bicategory/Functor/Lax.lean,Mathlib/CategoryTheory/Bicategory/Functor/Oplax.lean,Mathlib/CategoryTheory/Bicategory/Functor/Prelax.lean,Mathlib/CategoryTheory/Bicategory/Functor/Pseudofunctor.lean,Mathlib/CategoryTheory/Bicategory/Functor/Strict.lean,Mathlib/CategoryTheory/Bicategory/Grothendieck.lean,Mathlib/CategoryTheory/Bicategory/LocallyDiscrete.lean,Mathlib/CategoryTheory/FiberedCategory/Grothendieck.lean |
8 |
4 |
['github-actions', 'joelriou', 'mathlib-bors', 'mathlib4-dependent-issues-bot'] |
nobody |
4-76351 4 days ago |
4-76352 4 days ago |
6-80397 6 days |
28384 |
euprunin author:euprunin |
chore(Algebra/Order/Ring): golf entire `cast_natAbs` |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
awaiting-author
label:t-algebra$ |
1/4 |
Mathlib/Algebra/Order/Ring/Cast.lean |
1 |
2 |
['github-actions', 'riccardobrasca'] |
riccardobrasca assignee:riccardobrasca |
4-75822 4 days ago |
4-75822 4 days ago |
25-31928 25 days |
28385 |
euprunin author:euprunin |
chore(Algebra/BigOperators/Finsupp): deprecate `Finsupp.sum_sum_index'` |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
awaiting-author
label:t-algebra$ |
1/4 |
Mathlib/Algebra/BigOperators/Finsupp/Basic.lean |
1 |
7 |
['euprunin', 'github-actions', 'riccardobrasca'] |
riccardobrasca assignee:riccardobrasca |
4-75799 4 days ago |
4-75799 4 days ago |
25-31871 25 days |
27701 |
vihdzp author:vihdzp |
feat: `a < b + c ↔ a < b ∨ ∃ d < c, a = b + d` |
...and analogous results on `CanonicallyOrderedAdd`.
---
- [x] depends on: #29084
[](https://gitpod.io/from-referrer/)
|
t-algebra
awaiting-author
label:t-algebra$ |
41/0 |
Mathlib/Algebra/Order/Monoid/Canonical/Basic.lean |
1 |
5 |
['YaelDillies', 'github-actions', 'mathlib4-dependent-issues-bot', 'vihdzp'] |
nobody |
4-75045 4 days ago |
4-75085 4 days ago |
0-42619 11 hours |
26881 |
emo916math author:emo916math |
feat(Analysis/Calculus/Deriv/Star) A formula for `deriv (conj ∘ f ∘ conj)` |
Added a lemma that `deriv (conj ∘ f ∘ conj) = conj ∘ deriv f ∘ conj`, proved by cases on whether the derivative mathematically exists or not. This PR replaces [#26805](https://github.com/leanprover-community/mathlib4/pull/26805); see discussion there.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-analysis
awaiting-author
|
50/2 |
Mathlib/Analysis/Calculus/Deriv/Star.lean |
1 |
15 |
['emo916math', 'github-actions', 'j-loreaux', 'kckennylau'] |
j-loreaux assignee:j-loreaux |
4-68994 4 days ago |
35-68548 1 month ago |
31-70593 31 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
awaiting-author
|
31/0 |
Mathlib/Data/ULift.lean |
1 |
23 |
['eric-wieser', 'github-actions', 'grunweg', 'robertmaxton42'] |
nobody |
4-66803 4 days ago |
16-10418 16 days ago |
118-2181 118 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$ |
219/10 |
Mathlib.lean,Mathlib/Algebra/Algebra/Bilinear.lean,Mathlib/Algebra/Algebra/Defs.lean,Mathlib/LinearAlgebra/TensorProduct/Basic.lean,Mathlib/RingTheory/Coalgebra/Basic.lean,Mathlib/RingTheory/Coalgebra/Convolution.lean,Mathlib/RingTheory/Regular/RegularSequence.lean |
7 |
76 |
['YaelDillies', 'erdOne', 'eric-wieser', 'github-actions', 'kbuzzard', 'smorel394', 'themathqueen'] |
kbuzzard assignee:kbuzzard |
4-65444 4 days ago |
16-3655 16 days ago |
110-56107 110 days |
29437 |
NotWearingPants author:NotWearingPants |
feat(Data/Seq): add Seq.subsequence and prove basic theorems about it |
I added `Seq.subsequence` to compose a sequence with a monotone function, creating a subsequence. Aliased to `Seq.comp` since it's a composition.
I also added `Nat.le_induction_step_iff` which is needed to prove a subsequence is a sequence. This proves the comment at the top of `Defs.lean` that says "if `f n = none`, then `f m = none` for all `m ≥ n`" while `IsSeq` only talks about `n+1`.
For completion I added the same statement for `Int`.
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-data
new-contributor
|
115/1 |
Mathlib/Data/Int/Init.lean,Mathlib/Data/Nat/Init.lean,Mathlib/Data/Seq/Basic.lean,Mathlib/Data/Seq/Defs.lean |
4 |
1 |
['github-actions'] |
nobody |
4-61966 4 days ago |
4-84631 4 days ago |
4-84675 4 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/)
|
t-data
new-contributor
|
31/0 |
Mathlib.lean,Mathlib/Data/PNat/Order.lean |
2 |
14 |
['Ruben-VandeVelde', 'eric-wieser', 'github-actions', 'jburroni', 'vihdzp'] |
ericrbg assignee:ericrbg |
4-60785 4 days ago |
4-65789 4 days ago |
74-68103 74 days |
26330 |
Timeroot author:Timeroot |
feat: "Junk value" test file |
This PR continues the work from #25173.
Original PR: https://github.com/leanprover-community/mathlib4/pull/25173 |
t-data |
360/0 |
MathlibTest/Junk.lean |
1 |
8 |
['NotWearingPants', 'Timeroot', 'bryangingechen', 'github-actions', 'leanprover-community-bot-assistant', 'madvorak', 'vihdzp'] |
nobody |
4-59060 4 days ago |
64-51397 2 months ago |
80-13876 80 days |
29439 |
themathqueen author:themathqueen |
feat(Analysis/InnerProductSpace/Projection/Basic): `e ∘ f = 0` iff `(ker e).starProjection ∘ f = f` |
---
[](https://gitpod.io/from-referrer/)
|
t-analysis |
13/0 |
Mathlib/Analysis/InnerProductSpace/Projection/Basic.lean |
1 |
1 |
['github-actions'] |
nobody |
4-58114 4 days ago |
4-68181 4 days ago |
4-68221 4 days |
29435 |
sgouezel author:sgouezel |
WIP: typeclass experiment |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
WIP
label:t-algebra$ |
33/7 |
Mathlib/Algebra/QuadraticAlgebra.lean,Mathlib/Algebra/Ring/Defs.lean,Mathlib/GroupTheory/GroupAction/Hom.lean |
3 |
5 |
['eric-wieser', 'github-actions', 'leanprover-bot', 'sgouezel'] |
nobody |
4-57226 4 days ago |
5-1864 5 days ago |
0-1 1 second |
28945 |
harahu author:harahu |
doc: hyphenate compound adjectives ending in -dimensional |
Compound adjectives appearing before the noun they are modifying should be hyphenated in order to avoid ambiguity. This PR hyphenates such compound adjectives than are ending in "-dimensional".
It does not cover similar compound adjectives appearing _after_ their noun, as hyphenation is then regarded as a stylistic choice, as opposed to a grammatical tool.
---
[](https://gitpod.io/from-referrer/)
|
maintainer-merge |
180/180 |
Mathlib/Algebra/Azumaya/Matrix.lean,Mathlib/Algebra/BrauerGroup/Defs.lean,Mathlib/Algebra/Category/FGModuleCat/Basic.lean,Mathlib/Algebra/Category/FGModuleCat/Limits.lean,Mathlib/Algebra/Lie/Derivation/Killing.lean,Mathlib/Algebra/Lie/Weights/RootSystem.lean,Mathlib/Algebra/Module/ZLattice/Basic.lean,Mathlib/Algebra/Module/ZLattice/Covolume.lean,Mathlib/Analysis/BoundedVariation.lean,Mathlib/Analysis/Calculus/BumpFunction/Basic.lean,Mathlib/Analysis/Calculus/BumpFunction/SmoothApprox.lean,Mathlib/Analysis/Calculus/ContDiff/FiniteDimension.lean,Mathlib/Analysis/Calculus/Deriv/AffineMap.lean,Mathlib/Analysis/Calculus/Implicit.lean,Mathlib/Analysis/Calculus/LineDeriv/QuadraticMap.lean,Mathlib/Analysis/Complex/AbsMax.lean,Mathlib/Analysis/Complex/Tietze.lean,Mathlib/Analysis/Convex/AmpleSet.lean,Mathlib/Analysis/Convex/Continuous.lean,Mathlib/Analysis/Convex/Measure.lean,Mathlib/Analysis/Convex/SimplicialComplex/Basic.lean,Mathlib/Analysis/Distribution/AEEqOfIntegralContDiff.lean,Mathlib/Analysis/FunctionalSpaces/SobolevInequality.lean,Mathlib/Analysis/InnerProductSpace/Adjoint.lean,Mathlib/Analysis/InnerProductSpace/EuclideanDist.lean,Mathlib/Analysis/InnerProductSpace/JointEigenspace.lean,Mathlib/Analysis/InnerProductSpace/PiL2.lean,Mathlib/Analysis/InnerProductSpace/Spectrum.lean,Mathlib/Analysis/Normed/Module/FiniteDimension.lean,Mathlib/Analysis/Normed/Operator/ContinuousLinearMap.lean,Mathlib/Analysis/NormedSpace/HahnBanach/Extension.lean,Mathlib/Analysis/RCLike/Lemmas.lean,Mathlib/CategoryTheory/Preadditive/Schur.lean,Mathlib/Combinatorics/Additive/AP/Three/Behrend.lean,Mathlib/FieldTheory/Differential/Liouville.lean,Mathlib/FieldTheory/IntermediateField/Algebraic.lean,Mathlib/FieldTheory/IsAlgClosed/Spectrum.lean,Mathlib/FieldTheory/PrimitiveElement.lean,Mathlib/FieldTheory/PurelyInseparable/Basic.lean,Mathlib/Geometry/Manifold/BumpFunction.lean,Mathlib/Geometry/Manifold/ChartedSpace.lean,Mathlib/Geometry/Manifold/Diffeomorph.lean,Mathlib/Geometry/Manifold/Metrizable.lean,Mathlib/Geometry/Manifold/PartitionOfUnity.lean,Mathlib/LinearAlgebra/Coevaluation.lean,Mathlib/LinearAlgebra/Complex/FiniteDimensional.lean,Mathlib/LinearAlgebra/Complex/Module.lean,Mathlib/LinearAlgebra/Dimension/Finite.lean,Mathlib/LinearAlgebra/Dimension/Finrank.lean,Mathlib/LinearAlgebra/Dimension/FreeAndStrongRankCondition.lean,Mathlib/LinearAlgebra/FiniteDimensional/Basic.lean,Mathlib/LinearAlgebra/FiniteDimensional/Defs.lean,Mathlib/LinearAlgebra/FiniteDimensional/Lemmas.lean,Mathlib/LinearAlgebra/Matrix/FiniteDimensional.lean,Mathlib/LinearAlgebra/Matrix/GeneralLinearGroup/Card.lean,Mathlib/LinearAlgebra/Multilinear/FiniteDimensional.lean,Mathlib/MeasureTheory/Integral/TorusIntegral.lean,Mathlib/MeasureTheory/Measure/Haar/InnerProductSpace.lean,Mathlib/MeasureTheory/Measure/Haar/OfBasis.lean,Mathlib/MeasureTheory/Measure/Lebesgue/EqHaar.lean,Mathlib/MeasureTheory/Measure/Lebesgue/VolumeOfBalls.lean,Mathlib/Order/RelSeries.lean,Mathlib/Probability/Process/FiniteDimensionalLaws.lean,Mathlib/RepresentationTheory/FDRep.lean,Mathlib/RepresentationTheory/Maschke.lean,Mathlib/RepresentationTheory/Tannaka.lean,Mathlib/RingTheory/Finiteness/Basic.lean,Mathlib/RingTheory/Finiteness/Lattice.lean,Mathlib/RingTheory/Grassmannian.lean,Mathlib/Tactic/FunProp/Theorems.lean,Mathlib/Topology/Algebra/InfiniteSum/Defs.lean,Mathlib/Topology/Algebra/Module/FiniteDimension.lean,Mathlib/Topology/MetricSpace/HausdorffDimension.lean,MathlibTest/fun_prop.lean,docs/overview.yaml,docs/undergrad.yaml |
76 |
6 |
['github-actions', 'mathlib4-merge-conflict-bot', 'tb65536'] |
tb65536 assignee:tb65536 |
4-51885 4 days ago |
4-51904 4 days ago |
17-46089 17 days |
29420 |
llllvvuu author:llllvvuu |
chore: golf `LinearMap.charpoly_toMatrix` and add corollaries |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
31/39 |
Mathlib/LinearAlgebra/Charpoly/ToMatrix.lean |
1 |
1 |
['github-actions'] |
nobody |
4-49356 4 days ago |
5-33182 5 days ago |
5-33229 5 days |
28967 |
utkuokur author:utkuokur |
refactor(Combinatorics/SimpleGraph/Walk): simplify proof of "support_tail_of_not_nil" |
The proof of the lemma named "support_tail_of_not_nil" is shortened. Since "support_tail" is not needed anymore, it is removed.
@[deprecated (since := "2025-08-26")] sign is added for the removed "support_tail".
The library references to "support_tail" are replaced with "support_tail_of_not_nil".
To keep [@simp] on "cons_support_tail" and avoid the linter error, the [@simp] of "support_tail_of_not_nil" (previously on "support_tail") is removed. There might be a better way that I am missing, to deal with the linter error.
---
Additionally, a merge conflict with `master` was resolved by keeping the
generalized `support_tail_of_not_nil` and reintroducing `support_tail` as
a deprecated alias for compatibility.
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-combinatorics
|
7/10 |
Mathlib/Combinatorics/SimpleGraph/Hamiltonian.lean,Mathlib/Combinatorics/SimpleGraph/Walk.lean |
2 |
3 |
['github-actions', 'mathlib4-merge-conflict-bot', 'themathqueen'] |
awainverse assignee:awainverse |
4-49236 4 days ago |
4-50052 4 days ago |
17-65969 17 days |
29448 |
j-loreaux author:j-loreaux |
chore(Analysis/{NormedSpace/ConformalLinearMap → Normed/Operator/Conformal}): move file |
This is part of #28698 to migrate the material in `Analysis/NormedSpace/` to other locations.
---
[](https://gitpod.io/from-referrer/)
|
file-removed
tech debt
t-analysis
|
3/3 |
Mathlib.lean,Mathlib/Analysis/Calculus/Conformal/NormedSpace.lean,Mathlib/Analysis/InnerProductSpace/ConformalLinearMap.lean,Mathlib/Analysis/Normed/Operator/Conformal.lean |
4 |
1 |
['github-actions'] |
nobody |
4-45986 4 days ago |
4-45986 4 days ago |
4-46030 4 days |
26282 |
AntoineChambert-Loir author:AntoineChambert-Loir |
feat: a theorem of Jordan on primitive subgroups of the permutation group |
A theorem of Jordan on the primitive subgroups of a permutation group:
* if it contains a swap, it is equal to the permutation group,
* if it contains a 3-cycle, it contains the alternating group.
This PR continues the work from #24131.
---
- [x] depends on: #26281
- [x] depends on: #26280
- [x] depends on: #26279
Original PR: https://github.com/leanprover-community/mathlib4/pull/24131
[](https://gitpod.io/from-referrer/) |
t-group-theory
large-import
|
951/137 |
Mathlib.lean,Mathlib/Data/Set/Card.lean,Mathlib/GroupTheory/GroupAction/FixingSubgroup.lean,Mathlib/GroupTheory/GroupAction/Jordan.lean,Mathlib/GroupTheory/GroupAction/MultiplePrimitivity.lean,Mathlib/GroupTheory/GroupAction/MultipleTransitivity.lean,Mathlib/GroupTheory/GroupAction/Primitive.lean,Mathlib/GroupTheory/GroupAction/SubMulAction/OfFixingSubgroup.lean,Mathlib/GroupTheory/GroupAction/SubMulAction/OfStabilizer.lean,Mathlib/GroupTheory/Perm/Cycle/Type.lean,Mathlib/SetTheory/Cardinal/Embedding.lean |
11 |
n/a |
['AntoineChambert-Loir', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'tb65536'] |
nobody |
4-45396 4 days ago |
unknown |
unknown |
29351 |
staroperator author:staroperator |
feat(SetTheory/Cardinal): generalize and rename theorems on `Cardinal.sum` |
Some theorems on `Cardinal.sum f` are taking `f : ι → Cardinal.{max u v}`, which can be generalized to `f : ι → Cardinal.{v}`. Also rename `sum_le_iSup_lift`, `sum_lt_lift_of_isRegular`, `sum_eq_iSup_lift` etc. to reflect their signatures in names.
---
[](https://gitpod.io/from-referrer/)
|
t-set-theory |
79/36 |
Mathlib/Data/W/Cardinal.lean,Mathlib/ModelTheory/Encoding.lean,Mathlib/SetTheory/Cardinal/Arithmetic.lean,Mathlib/SetTheory/Cardinal/Basic.lean,Mathlib/SetTheory/Cardinal/Cofinality.lean,Mathlib/SetTheory/Cardinal/Defs.lean,Mathlib/SetTheory/Cardinal/Order.lean,Mathlib/SetTheory/Cardinal/Ordinal.lean,Mathlib/SetTheory/Cardinal/Pigeonhole.lean,Mathlib/SetTheory/Cardinal/Regular.lean |
10 |
5 |
['github-actions', 'staroperator', 'vihdzp'] |
nobody |
4-41072 4 days ago |
8-40971 8 days ago |
8-60163 8 days |
29429 |
kim-em author:kim-em |
feat: `grind` annotations for `Finset.card` |
---
[](https://gitpod.io/from-referrer/)
|
t-data |
161/162 |
Archive/Imo/Imo1998Q2.lean,Counterexamples/AharoniKorman.lean,Mathlib/Algebra/BigOperators/Ring/Finset.lean,Mathlib/Combinatorics/Additive/PluenneckeRuzsa.lean,Mathlib/Combinatorics/Hall/Finite.lean,Mathlib/Combinatorics/SetFamily/Compression/UV.lean,Mathlib/Combinatorics/SetFamily/HarrisKleitman.lean,Mathlib/Combinatorics/SetFamily/KruskalKatona.lean,Mathlib/Combinatorics/SetFamily/Shadow.lean,Mathlib/Combinatorics/SimpleGraph/DeleteEdges.lean,Mathlib/Combinatorics/SimpleGraph/Extremal/Turan.lean,Mathlib/Combinatorics/SimpleGraph/Finite.lean,Mathlib/Combinatorics/SimpleGraph/FiveWheelLike.lean,Mathlib/Combinatorics/SimpleGraph/Operations.lean,Mathlib/Combinatorics/SimpleGraph/Regularity/Chunk.lean,Mathlib/Combinatorics/SimpleGraph/Regularity/Equitabilise.lean,Mathlib/Combinatorics/SimpleGraph/StronglyRegular.lean,Mathlib/Combinatorics/SimpleGraph/Triangle/Basic.lean,Mathlib/Combinatorics/SimpleGraph/Triangle/Counting.lean,Mathlib/Data/Finset/Card.lean,Mathlib/Data/Finset/CastCard.lean,Mathlib/Data/Finset/Insert.lean,Mathlib/Data/Finset/Interval.lean,Mathlib/Data/Finset/Lattice/Lemmas.lean,Mathlib/Data/Fintype/Card.lean,Mathlib/Data/Nat/Totient.lean,Mathlib/Data/Set/Card/Arithmetic.lean,Mathlib/Geometry/Euclidean/Circumcenter.lean,Mathlib/LinearAlgebra/Lagrange.lean,Mathlib/LinearAlgebra/Multilinear/Basic.lean,Mathlib/NumberTheory/JacobiSum/Basic.lean,Mathlib/Order/Interval/Finset/Box.lean |
32 |
2 |
['github-actions', 'grunweg'] |
nobody |
4-40180 4 days ago |
5-17249 5 days ago |
5-17288 5 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).
Co-authored by:
- [Viviana del Barco](https://github.com/vdelbarc)
- [Gustavo Infanti](https://github.com/GuQOliveira)
- [Exequiel Rivas](https://github.com/erivas)
---
I am not sure whether the `prodEquivOfIsCompl_symm_apply` theorem should be tagged with `@[simp]`; this might lead to confluence issues. Opinions are welcome!
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-algebra
awaiting-author
label:t-algebra$ |
10/0 |
Mathlib/LinearAlgebra/Projection.lean |
1 |
7 |
['PSchwahn', 'github-actions', 'joelriou', 'kckennylau'] |
joelriou assignee:joelriou |
4-39063 4 days ago |
4-70166 4 days ago |
73-43225 73 days |
29398 |
vihdzp author:vihdzp |
feat: `Polynomial.coeffs_nonempty_iff` |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
easy
label:t-algebra$ |
4/0 |
Mathlib/Algebra/Polynomial/Basic.lean |
1 |
3 |
['Ruben-VandeVelde', 'github-actions', 'vihdzp'] |
nobody |
4-37235 4 days ago |
6-2873 6 days ago |
6-2861 6 days |
29454 |
kim-em author:kim-em |
feat: `grind` annotations for `Nat.count` |
---
[](https://gitpod.io/from-referrer/)
|
|
16/20 |
Mathlib/Algebra/Group/Embedding.lean,Mathlib/Data/Nat/Count.lean |
2 |
1 |
['github-actions'] |
nobody |
4-36410 4 days ago |
4-36483 4 days ago |
4-36464 4 days |
29455 |
kim-em author:kim-em |
chore: grind annotations in Data/Nat/Find |
---
[](https://gitpod.io/from-referrer/)
|
t-data |
5/3 |
Mathlib/Data/Nat/Find.lean |
1 |
1 |
['github-actions'] |
nobody |
4-35911 4 days ago |
4-35926 4 days ago |
4-35963 4 days |
29133 |
ScottCarnahan author:ScottCarnahan |
chore (Algebra/Vertex): linearize coefficient functions |
This PR upgrades the coefficient functions of vertex operators and heterogeneous vertex operators to be linear maps instead of just functions. We also deprecate the corresponding linearity lemmas, and add two rfl simp lemmas.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
40/44 |
Mathlib/Algebra/Vertex/HVertexOperator.lean,Mathlib/Algebra/Vertex/VertexOperator.lean |
2 |
1 |
['github-actions'] |
riccardobrasca assignee:riccardobrasca |
4-34917 4 days ago |
13-84407 13 days ago |
13-84446 13 days |
29154 |
ScottCarnahan author:ScottCarnahan |
feat (Algebra/Lie): Define low-degree cochains and differentials for coefficients with trivial action |
This PR defines 1-cochains and 2-cochains of a Lie algebra `L` with coefficients in a module `M` on which `L` acts trivially. This special case is useful for constructing central extensions of Lie algebras, while not needing the general machinery of Lie algebra cohomology.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
143/0 |
Mathlib.lean,Mathlib/Algebra/Lie/Basic.lean,Mathlib/Algebra/Lie/CochainTrivial.lean |
3 |
1 |
['github-actions'] |
mariainesdff assignee:mariainesdff |
4-34916 4 days ago |
13-18842 13 days ago |
13-18878 13 days |
29224 |
euprunin author:euprunin |
chore: remove redundant `rcases` invocations |
---
**Note:** Although technically redundant, some of these may be worth keeping for readability, or other reasons. Let me know if you think any should stay.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
1/10 |
Mathlib/Algebra/Algebra/Defs.lean,Mathlib/Algebra/Group/Ext.lean,Mathlib/Algebra/Module/Injective.lean,Mathlib/Algebra/Polynomial/Basic.lean,Mathlib/Algebra/Polynomial/Coeff.lean,Mathlib/Algebra/Polynomial/Degree/Definitions.lean,Mathlib/Algebra/Polynomial/Degree/Support.lean |
7 |
4 |
['github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot'] |
chrisflav assignee:chrisflav |
4-34913 4 days ago |
11-41402 11 days ago |
11-53453 11 days |
29456 |
kim-em author:kim-em |
chore: basic grind annotations for Real.sqrt |
---
[](https://gitpod.io/from-referrer/)
|
|
16/10 |
Mathlib/Data/Real/Sqrt.lean,Mathlib/Order/Defs/LinearOrder.lean |
2 |
1 |
['github-actions'] |
nobody |
4-33201 4 days ago |
4-33270 4 days ago |
4-33251 4 days |
29449 |
mitchell-horner author:mitchell-horner |
feat(Combinatorics/SimpleGraph): add Turán density related theorems |
Refactors `tendsto_turanDensity` and implements `turanDensity_eq_sInf` and `isContained_of_card_edgeFinset` (theorems that are common in proofs involving Turán density).
---
[](https://gitpod.io/from-referrer/)
|
t-combinatorics |
52/14 |
Mathlib/Combinatorics/SimpleGraph/Extremal/TuranDensity.lean |
1 |
1 |
['github-actions'] |
nobody |
4-29268 4 days ago |
4-44663 4 days ago |
4-44707 4 days |
29458 |
LiamSchilling author:LiamSchilling |
feat(MvPolynomial/WeightedHomogenous): relate `weightedTotalDegree` to `degrees`, `totalDegree`, and `degreeOf` |
`weightedTotalDegree` is the most general notion of multivariate degree in mathlib. These theorems show that it specializes to `degrees`, `totalDegree`, and `degreeOf` with specialized weights.
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
new-contributor
|
24/1 |
Mathlib/RingTheory/MvPolynomial/WeightedHomogeneous.lean |
1 |
1 |
['github-actions'] |
nobody |
4-20789 4 days ago |
4-20806 4 days ago |
4-20843 4 days |
28248 |
YaelDillies author:YaelDillies |
feat: expectation and (conditional) variance of a Bernoulli random variable |
Compute the expectation, variance, conditional variance of a Bernoulli random variable.
From MiscYD
---
[](https://gitpod.io/from-referrer/)
|
t-measure-probability
awaiting-author
|
240/0 |
Mathlib.lean,Mathlib/MeasureTheory/Integral/Bochner/Set.lean,Mathlib/MeasureTheory/Measure/MeasureSpaceDef.lean,Mathlib/Probability/Bernoulli.lean,Mathlib/Probability/HasLaw.lean,Mathlib/Probability/Moments/Variance.lean |
6 |
34 |
['DavidLedvinka', 'RemyDegenne', 'YaelDillies', 'github-actions', 'kex-y', 'pfaffelh', 'themathqueen'] |
kex-y assignee:kex-y |
4-12615 4 days ago |
4-12615 4 days ago |
28-39091 28 days |
29434 |
ntapiam author:ntapiam |
feat(NonAssoc/LieAdmissible): prove every ring/algebra is LieAdmissible |
-awaiting-author |
new-contributor
t-algebra
label:t-algebra$ |
27/6 |
Mathlib/Algebra/NonAssoc/LieAdmissible/Defs.lean |
1 |
1 |
['github-actions'] |
nobody |
4-10442 4 days ago |
5-3218 5 days ago |
5-3261 5 days |
26735 |
Raph-DG author:Raph-DG |
feat(AlgebraicGeometry): The codimension of a point of a scheme is equal to the krull dimension of the stalk |
In this PR we show that the codimension of a point in a scheme is equal to the krull dimension of the local ring at that point, as in stacks 02IZ.
---
The proof of the main result `stalk_dim_eq_coheight` is currently a bit long for my (and I suspect the broader community's) tastes. That said, I'm not quite sure the best way to break it into pieces, any comments would be very much appreciated!
- [x] depends on: #26204 [For the notion of codimension, here we are using the coheight in the specialization order. ]
- [ ] depends on: #26225
[](https://gitpod.io/from-referrer/)
|
t-algebraic-geometry |
204/1 |
Mathlib/AlgebraicGeometry/Properties.lean,Mathlib/Order/KrullDimension.lean,Mathlib/Topology/KrullDimension.lean |
3 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
4-9950 4 days ago |
4-11192 4 days ago |
4-11966 4 days |
29459 |
bwangpj author:bwangpj |
feat: ContMDiffAt.pow |
Powers of `C^n` functions `M → G` into a commutative monoid `G` are `C^n`.
This is upstreamed from [https://github.com/girving/ray](https://github.com/girving/ray).
Co-authored-by: Geoffrey Irving
---
[](https://gitpod.io/from-referrer/)
|
maintainer-merge
t-differential-geometry
|
20/2 |
Mathlib/Geometry/Manifold/Algebra/Monoid.lean |
1 |
4 |
['github-actions', 'grunweg'] |
grunweg assignee:grunweg |
4-6989 4 days ago |
4-7202 4 days ago |
4-17627 4 days |
28908 |
joelriou author:joelriou |
feat(CategoryTheory): Pullback functors on `Over` categories in `Type` have right adjoints |
Given a map `f : E → B`, in order to show that `Over.pullback f : Over B ⥤ Over E` commutes with colimits, we show that it admits a right adjoint. In order to do that, we first construct a functor `overPullback f : Over B ⥤ Over E` whose definition involves explicit types rather than categorical pullbacks, and we define its right adjoint `overPushforward f : Over E ⥤ Over B`.
(In a future PR, it will be shown that the `Over.pullback` also commutes with colimits in categories of presheaves, and hopefully this will be used in the construction of the Quillen model category structure on simplicial sets.)
---
[](https://gitpod.io/from-referrer/)
|
t-category-theory
awaiting-author
|
103/0 |
Mathlib.lean,Mathlib/CategoryTheory/Limits/Types/OverPullback.lean,Mathlib/CategoryTheory/Limits/Types/Shapes.lean |
3 |
9 |
['emilyriehl', 'github-actions', 'joelriou', 'mathlib4-merge-conflict-bot', 'robin-carlier', 'sinhp'] |
nobody |
4-751 4 days ago |
4-77366 4 days ago |
13-55990 13 days |
27162 |
themathqueen author:themathqueen |
feat(Analysis/InnerProductSpace/Positive): `U.starProjection ≤ V.starProjection` iff `U ≤ V` |
For symmetric projections `p` and `q`, `p ≤ q` iff `q ∘ p = p`, so then: `U.starProjection ≤ V.starProjection` iff `U ≤ V`, which implies that `Submodule.starProjection` is an injective function.
---
- [x] depends on: #25910
- [x] depends on: #27619
- [x] depends on: #27642
[](https://gitpod.io/from-referrer/)
|
t-analysis |
58/0 |
Mathlib/Analysis/InnerProductSpace/Positive.lean,Mathlib/Analysis/InnerProductSpace/Symmetric.lean |
2 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
j-loreaux assignee:j-loreaux |
3-85737 3 days ago |
24-42864 24 days ago |
29-23290 29 days |
28533 |
kim-em author:kim-em |
feat(linarith): add `linarith?` mode which suggests a `linarith only` call |
Adds `linarith?`, which traces the internal to watch which inequalities are being used, and suggests a `linarith only` call via the "try this:" mechanism.
Also adds a `+minimize` flag, on by default, which then greedily tries to drop hypotheses from the used set, to see if the problem is still possible with a smaller set. Currently I don't have test case showing this is worthwhile, however. Contributions welcome.
------
https://chatgpt.com/codex/tasks/task_e_68a02bce93a883218485c7e7cafb877a |
codex
t-meta
|
212/68 |
Mathlib/Tactic/Linarith/Frontend.lean,Mathlib/Tactic/Linarith/Verification.lean,MathlibTest/linarith.lean |
3 |
8 |
['YaelDillies', 'github-actions', 'hrmacbeth', 'jcommelin', 'kim-em', 'mathlib4-merge-conflict-bot'] |
robertylewis assignee:robertylewis |
3-83516 3 days ago |
11-27428 11 days ago |
27-26791 27 days |
28393 |
tristan-f-r author:tristan-f-r |
chore(WithZero): clean |
We replace `erw` this with defeq abuse (which seems to be accepted as okay inside proofs), and clean up the rest of the file.
I might start trying to remove `erw`s in Mathlib.
---
[](https://gitpod.io/from-referrer/)
|
t-data
awaiting-author
|
14/16 |
Mathlib/Data/Int/WithZero.lean |
1 |
10 |
['Ruben-VandeVelde', 'github-actions', 'ocfnash', 'tristan-f-r'] |
nobody |
3-78922 3 days ago |
3-78922 3 days ago |
26-24564 26 days |
29470 |
NotWearingPants author:NotWearingPants |
chore(Algebra/Group/Action/Faithful): fix typo in LefttCancelMonoid |
chore(Algebra/Group/Action/Faithful): fix typo in LefttCancelMonoid
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-algebra
easy
label:t-algebra$ |
1/1 |
Mathlib/Algebra/Group/Action/Faithful.lean |
1 |
2 |
['NotWearingPants', 'github-actions'] |
nobody |
3-72515 3 days ago |
3-72519 3 days ago |
3-72557 3 days |
28950 |
Vierkantor author:Vierkantor |
fix(TacticAnalysis): comment out syntax range check |
In #28802 we discovered the tactic analysis framework does not fire on declarations using `where` clauses. The reason is that `def foo where ...` gets turned into `def foo := { ... }`, and the `{ ... }` syntax is assigned a range outside of the `where ...` syntax; this causes the syntax range check to omit the whole declaration body. I am not entirely sure this is a bug in Lean or it was a misuse of ranges; in the meantime it should be okay to skip the check: the worst that happens is we analyze a piece of syntax outside of the declaration, which we'd get to later anyway.
---
[](https://gitpod.io/from-referrer/)
|
t-meta |
23/3 |
Mathlib/Tactic/TacticAnalysis.lean,MathlibTest/TacticAnalysis.lean |
2 |
3 |
['Vierkantor', 'github-actions', 'thorimur'] |
robertylewis assignee:robertylewis |
3-70633 3 days ago |
18-2969 18 days ago |
18-2951 18 days |
26211 |
Thmoas-Guan author:Thmoas-Guan |
feat(Algebra): vanishing of induced hom between ext |
In this PR we proved that the map `Ext(N,M)` -> `Ext(N,M)` induced by left scalar multiplication with `x` on `M` is zero for `x` in `ann(N)`.
Co-authored-by: Wang Jingting
Co-authored-by: Hu Yongle
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebra
label:t-algebra$ |
88/3 |
Mathlib/RingTheory/Ideal/AssociatedPrime/Localization.lean,Mathlib/RingTheory/Regular/Category.lean,Mathlib/RingTheory/Regular/Depth.lean |
3 |
n/a |
['Thmoas-Guan', 'github-actions'] |
nobody |
3-68035 3 days ago |
unknown |
unknown |
26210 |
Thmoas-Guan author:Thmoas-Guan |
feat(RingTheory): associated primes of localized module |
We prove that `Ass(S^{-1}M)` is equal to the preimage of `Ass(M)` under `Ideal.comap` if the base ring is Noetherian.
From this we conclude that every minimal prime over `Module.annihilator R M` is in `Ass(M)` when `M` is finitely generated.
---
[](https://gitpod.io/from-referrer/) |
t-ring-theory
large-import
awaiting-author
|
85/22 |
Mathlib/RingTheory/Ideal/AssociatedPrime/Localization.lean,Mathlib/RingTheory/Regular/Depth.lean |
2 |
30 |
['Thmoas-Guan', 'chrisflav', 'github-actions', 'mathlib4-merge-conflict-bot', 'mbkybky'] |
chrisflav assignee:chrisflav |
3-67193 3 days ago |
18-28438 18 days ago |
36-71207 36 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-ring-theory
awaiting-author
|
241/15 |
Mathlib.lean,Mathlib/LinearAlgebra/Quotient/Basic.lean,Mathlib/RingTheory/Ideal/MinimalPrime/Localization.lean,Mathlib/RingTheory/Jacobson/Ideal.lean,Mathlib/RingTheory/KrullDimension/Module.lean,Mathlib/RingTheory/KrullDimension/Regular.lean,Mathlib/RingTheory/LocalRing/MaximalIdeal/Basic.lean,Mathlib/RingTheory/Nakayama.lean,Mathlib/RingTheory/Support.lean |
9 |
n/a |
['Thmoas-Guan', 'chrisflav', 'github-actions', 'leanprover-community-bot-assistant', 'mbkybky'] |
chrisflav assignee:chrisflav |
3-67089 3 days ago |
unknown |
unknown |
27567 |
themathqueen author:themathqueen |
feat(LinearAlgebra/TensorProduct/Associator): add `lid` and `assoc` tensor lemmas |
This adds `TensorProduct.lid_tensor` and `TensorProduct.assoc_tensor`.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
easy
label:t-algebra$ |
31/2 |
Mathlib/LinearAlgebra/TensorProduct/Associator.lean,Mathlib/LinearAlgebra/TensorProduct/Basic.lean |
2 |
3 |
['github-actions', 'themathqueen'] |
mattrobball assignee:mattrobball |
3-66969 3 days ago |
33-56492 1 month ago |
47-49326 47 days |
28097 |
themathqueen author:themathqueen |
feat(LinearAlgebra/Matrix/PosDef): kronecker of positive (semi-)definite matrices is positive (semi-)definite |
This first shows that `U * x * star U` is positive (semi-)definite if and only if `x` is, for an invertible matrix `U` in a not necessarily commutative star-ring. Then using the spectral theorem, it follows that the kronecker of positive (semi-)definite matrices is positive (semi-)definite.
---
- [x] depends on: #28093
- [x] depends on: #28476
- [x] depends on: #28544
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
67/6 |
Mathlib/Algebra/Star/SelfAdjoint.lean,Mathlib/LinearAlgebra/Matrix/Hermitian.lean,Mathlib/LinearAlgebra/Matrix/Kronecker.lean,Mathlib/LinearAlgebra/Matrix/PosDef.lean |
4 |
6 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'themathqueen'] |
nobody |
3-66442 3 days ago |
3-73480 3 days ago |
11-54836 11 days |
29383 |
Vierkantor author:Vierkantor |
chore(Topology): process porting notes |
Go through the porting notes in the Topology folder and solve the ones with an obvious fix.
This last batch of porting notes should bring us below 500 open porting notes in Mathlib, when the RingTheory ones get merged too!
---
[](https://gitpod.io/from-referrer/)
|
tech debt
t-topology
|
134/222 |
Mathlib/Topology/Algebra/Module/CharacterSpace.lean,Mathlib/Topology/Algebra/Monoid.lean,Mathlib/Topology/Algebra/MulAction.lean,Mathlib/Topology/Algebra/Ring/Ideal.lean,Mathlib/Topology/Bases.lean,Mathlib/Topology/Bornology/Basic.lean,Mathlib/Topology/Bornology/Constructions.lean,Mathlib/Topology/Category/Profinite/CofilteredLimit.lean,Mathlib/Topology/Category/TopCat/Limits/Basic.lean,Mathlib/Topology/Category/TopCat/Limits/Cofiltered.lean,Mathlib/Topology/Compactness/Compact.lean,Mathlib/Topology/Constructions/SumProd.lean,Mathlib/Topology/ContinuousMap/Periodic.lean,Mathlib/Topology/ContinuousMap/ZeroAtInfty.lean,Mathlib/Topology/DiscreteQuotient.lean,Mathlib/Topology/Gluing.lean,Mathlib/Topology/Homotopy/Basic.lean,Mathlib/Topology/Homotopy/Equiv.lean,Mathlib/Topology/Homotopy/HomotopyGroup.lean,Mathlib/Topology/LocallyConstant/Basic.lean,Mathlib/Topology/MetricSpace/Algebra.lean,Mathlib/Topology/MetricSpace/Equicontinuity.lean,Mathlib/Topology/MetricSpace/GromovHausdorff.lean,Mathlib/Topology/MetricSpace/IsometricSMul.lean,Mathlib/Topology/Order.lean,Mathlib/Topology/Order/Compact.lean,Mathlib/Topology/Separation/Basic.lean,Mathlib/Topology/Sheaves/CommRingCat.lean,Mathlib/Topology/Sheaves/SheafCondition/EqualizerProducts.lean,Mathlib/Topology/Sheaves/Sheafify.lean,Mathlib/Topology/Sheaves/Stalks.lean,Mathlib/Topology/UniformSpace/Cauchy.lean,Mathlib/Topology/UniformSpace/UniformConvergenceTopology.lean |
33 |
1 |
['github-actions'] |
nobody |
3-66219 3 days ago |
6-71690 6 days ago |
6-71672 6 days |
29475 |
euprunin author:euprunin |
chore(RingTheory/Extension/Presentation): remove use of `erw` in `aeval_comp_val_eq` |
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory |
0/1 |
Mathlib/RingTheory/Extension/Presentation/Basic.lean |
1 |
1 |
['github-actions'] |
nobody |
3-64177 3 days ago |
3-64185 3 days ago |
3-64229 3 days |
26909 |
gasparattila author:gasparattila |
feat(LinearAlgebra/Projectivization/Subspace): correspondence between linear and projective subspaces |
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-algebra
label:t-algebra$ |
69/3 |
Mathlib/LinearAlgebra/Projectivization/Subspace.lean |
1 |
5 |
['eric-wieser', 'gasparattila', 'github-actions'] |
Vierkantor assignee:Vierkantor |
3-59887 3 days ago |
66-52517 2 months ago |
66-52562 66 days |
29474 |
sgouezel author:sgouezel |
feat: explicit zsmul field in ring constructor to solve performance issue |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
2/0 |
Mathlib/Algebra/Ring/InjSurj.lean |
1 |
4 |
['github-actions', 'leanprover-bot', 'sgouezel'] |
nobody |
3-57384 3 days ago |
3-68246 3 days ago |
3-68281 3 days |
28175 |
dsfxcimk author:dsfxcimk |
feat: exterior angle theorem |
Add Exterior angle theorem
---
The Exterior Angle Theorem states that the exterior angle of a triangle equals the sum of the two non-adjacent interior angles.
I plan to place this in Mathlib.Geometry.Euclidean.Triangle
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-euclidean-geometry
awaiting-author
|
9/0 |
Mathlib/Geometry/Euclidean/Triangle.lean |
1 |
12 |
['FrankieNC', 'JovanGerb', 'dsfxcimk', 'github-actions', 'grunweg', 'mathlib4-merge-conflict-bot', 'themathqueen'] |
nobody |
3-55433 3 days ago |
3-77641 3 days ago |
28-57160 28 days |
28286 |
bwangpj author:bwangpj |
feat(Geometry/Manifold/ContMDiff): basic lemmas for analytic (`C^ω`) functions |
Add basic lemmas relating `ContMDiff` in the `C^ω` case to being `Analytic` on charts.
This is upstreamed from [https://github.com/girving/ray](https://github.com/girving/ray).
Co-authored-by: Geoffrey Irving
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-differential-geometry
awaiting-author
|
36/0 |
Mathlib/Geometry/Manifold/ContMDiff/Defs.lean |
1 |
13 |
['bwangpj', 'girving', 'github-actions', 'grunweg', 'kbuzzard', 'sgouezel'] |
sgouezel assignee:sgouezel |
3-53818 3 days ago |
4-7853 4 days ago |
27-76128 27 days |
28871 |
JaafarTanoukhi author:JaafarTanoukhi |
feat(Combinatorics/Digraph): Tournaments |
Define orientations and tournaments. Related to #26771.
Co-authored-by: Rida Hamadani
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-combinatorics
|
62/0 |
Mathlib.lean,Mathlib/Combinatorics/Digraph/Orientation.lean,Mathlib/Combinatorics/Digraph/Tournament.lean |
3 |
3 |
['JaafarTanoukhi', 'NotWearingPants', 'Rida-Hamadani', 'github-actions'] |
kmill assignee:kmill |
3-50617 3 days ago |
19-54803 19 days ago |
19-54842 19 days |
28793 |
grunweg author:grunweg |
feat: smooth immersions |
Define smooth immersions between manifolds.
We use a definition which allows for corners, infinite dimension and arbitrary fields.
Future PRs will
- prove that immersions are C^n (#28796),
- prove another characterisation of immersions: f is immersed at x iff the differential df_x splits,
i.e. is injective, has closed range and its image has a closed complement,
and in particular that a map between finite-dimensional manifolds over a complete field is an
immersion iff its differential is injective,
- use this to prove that the product (#28853) and composition of immersions is an immersion,
- use this theory to give more conceptual proofs of half of `Manifold/Instances/Icc.lean` (#29077)
- define smooth embeddings and immersed and embedded smooth submanifolds
---
- [x] depends on: #28701
Most of the above has been done at https://github.com/grunweg/mathlib4/tree/MR-define-immersions.
[](https://gitpod.io/from-referrer/)
|
t-differential-geometry |
275/4 |
Mathlib.lean,Mathlib/Geometry/Manifold/IsImmersionEmbedding.lean,docs/references.bib |
3 |
11 |
['chrisflav', 'github-actions', 'grunweg', 'mathlib4-dependent-issues-bot'] |
nobody |
3-50499 3 days ago |
4-50833 4 days ago |
4-53220 4 days |
25736 |
robin-carlier author:robin-carlier |
feat(AlgebraicTopology/SimplexCategory/GeneratorsRelations/NormalForms): Normal forms for `P_σ`s |
We prove that admissible lists introduced in #21744 indeed provide a suitable normal form for morphisms of `SimplexCategoryGenRel` satisfying `P_σ` (i.e that are compositions of degeneracies).
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, thanks to the fifth simplicial identity, composition on the right by some `σ i` corresponds to simplicial insertion of `i` in the list. This gives existence of a normal form for every morphism satisfying `P_σ`, i.e exhibits such morphism as some `standardσ`.
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. Since admissible lists are sorted, this fully characterizes the list, and thus shows that the list only depends on the morphism `standardσ` attached to it.
Part of a series of PR formalising that `SimplexCategoryGenRel` is equivalent to `SimplexCategory`.
---
- [x] depends on: #21744
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #21745.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/21745* |
t-algebraic-topology
large-import
|
189/7 |
Mathlib/AlgebraicTopology/SimplexCategory/GeneratorsRelations/NormalForms.lean |
1 |
12 |
['github-actions', 'jcommelin', 'joelriou', 'mathlib4-dependent-issues-bot', 'robin-carlier'] |
mattrobball assignee:mattrobball |
3-49311 3 days ago |
3-49366 3 days ago |
85-82730 85 days |
26824 |
robin-carlier author:robin-carlier |
feat(CategoryTheory/Monoidal/DayConvolution): Day functors type synonym |
Given monoidal categories `C` and `V`, we introduce a type synonym `DayFunctor C V` (denoted `C ⊛⥤ V`) for functors `C ⥤ V` and produce a category instance on it. Using the infrastructure from #26820, we show that this category admits a monoidal structure coming from Day convolution of functors. We provide a very basic API for this category, such as an abbreviation for the unit map of day convolutions, and a restatement of the universal property of the tensor product with respect to that unit.
---
- [x] depends on: #26820
[](https://gitpod.io/from-referrer/)
|
t-category-theory |
241/0 |
Mathlib.lean,Mathlib/CategoryTheory/Monoidal/DayConvolution/DayFunctor.lean |
2 |
n/a |
['github-actions', 'joelriou', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'robin-carlier'] |
nobody |
3-48997 3 days ago |
unknown |
unknown |
26614 |
Rida-Hamadani author:Rida-Hamadani |
feat(SimpleGraph): add more API for `take`/`drop` |
These came up while proving the Girth-Diameter inequality. The main lemma proves that taking `n` vertices of a walk results in a sub-walk of taking `k` vertices when `n` is less than or equal to `k`. The sub-walk relation is represented as `p.support.Sublist q.support` where `p` and `q` are walks.
- [ ] depends on: #26655
---
[](https://gitpod.io/from-referrer/)
|
t-combinatorics
awaiting-author
|
74/0 |
Mathlib/Combinatorics/SimpleGraph/Walk.lean |
1 |
18 |
['Rida-Hamadani', 'b-mehta', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
3-42696 3 days ago |
3-42728 3 days ago |
4-83551 4 days |
29118 |
edegeltje author:edegeltje |
chore(CategoryTheory): align `refl` and `rfl` declarations in CategoryTheory |
In general, theorems and declarations named `refl` take an explicit argument and prove/construct something of type `r X X`, whereas the `rfl` versions take the argument implicitly.
This PR adds missing `rfl` declarations to the CategoryTheory library, and makes sure `Equivalence.refl` takes an explicit argument.
---
[](https://gitpod.io/from-referrer/)
|
will-close-soon
t-category-theory
awaiting-author
|
37/18 |
Mathlib/CategoryTheory/Adjunction/Basic.lean,Mathlib/CategoryTheory/Enriched/Ordinary/Basic.lean,Mathlib/CategoryTheory/Equivalence.lean,Mathlib/CategoryTheory/IsConnected.lean,Mathlib/CategoryTheory/Iso.lean,Mathlib/CategoryTheory/Monoidal/Functor.lean,Mathlib/CategoryTheory/Retract.lean,Mathlib/CategoryTheory/Shift/Adjunction.lean,Mathlib/CategoryTheory/Sums/Products.lean,Mathlib/CategoryTheory/Triangulated/Adjunction.lean,Mathlib/RingTheory/Morita/Basic.lean |
11 |
6 |
['Ruben-VandeVelde', 'edegeltje', 'github-actions', 'joelriou'] |
TwoFX assignee:TwoFX |
3-41983 3 days ago |
3-41983 3 days ago |
11-13051 11 days |
29481 |
llllvvuu author:llllvvuu |
feat(LinearAlgebra/Eigenspace): roots of matrix minpoly give spectrum |
This is derived from the corresponding result on linear maps.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
28/0 |
Mathlib/LinearAlgebra/Eigenspace/Minpoly.lean |
1 |
2 |
['github-actions', 'llllvvuu'] |
nobody |
3-38038 3 days ago |
3-38064 3 days ago |
0-0 0 seconds |
28719 |
mitchell-horner author:mitchell-horner |
refactor: redefine `IsTuranMaximal` |
Redefined `IsTuranMaximal := G.IsExtremal (CliqueFree · (r + 1))` and
- replaced `classical` in `IsTuranMaximal.le_iff_eq` with `DecidableRel`
- refactored `turanGraph.instDecidableRelAdj`, `turanGraph_zero`, `exists_isTuranMaximal`
- added `open Fintype`
- replaced `simp only` with `rw` or `simp_rw`
---
- [x] depends on: #28721
- [x] depends on: #29054
[](https://gitpod.io/from-referrer/)
|
t-combinatorics |
33/46 |
Mathlib/Combinatorics/SimpleGraph/Extremal/Turan.lean |
1 |
7 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'mitchell-horner', 'vihdzp'] |
kmill assignee:kmill |
3-34905 3 days ago |
11-74216 11 days ago |
16-30910 16 days |
28987 |
euprunin author:euprunin |
chore(Analysis/Distribution): remove redundant `have` in `ae_eq_zero_of_integral_smooth_smul_eq_zero` |
---
[](https://gitpod.io/from-referrer/)
|
t-analysis |
0/2 |
Mathlib/Analysis/Distribution/AEEqOfIntegralContDiff.lean |
1 |
6 |
['euprunin', 'github-actions', 'grunweg', 'leanprover-bot', 'leanprover-community-mathlib4-bot'] |
hrmacbeth assignee:hrmacbeth |
3-34904 3 days ago |
10-45304 10 days ago |
10-47903 10 days |
29132 |
YaelDillies author:YaelDillies |
feat(AdjoinRoot): bundle operations as `AlgHom`s |
In particular, generalise and rename `liftHom` to use a general `eval₂` instead of `aeval`.
From Toric
Co-authored-by: Andrew Yang the.erd.one@gmail.com
Co-authored-by: Michał Mrugała kiolterino@gmail.com
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
toric
|
164/103 |
Mathlib/Algebra/Algebra/Hom.lean,Mathlib/FieldTheory/IntermediateField/Adjoin/Basic.lean,Mathlib/FieldTheory/Isaacs.lean,Mathlib/FieldTheory/KummerExtension.lean,Mathlib/FieldTheory/Minpoly/IsIntegrallyClosed.lean,Mathlib/RingTheory/Adjoin/Field.lean,Mathlib/RingTheory/AdjoinRoot.lean,Mathlib/RingTheory/LocalRing/ResidueField/Instances.lean,Mathlib/RingTheory/Localization/Away/AdjoinRoot.lean |
9 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
erdOne assignee:erdOne |
3-34902 3 days ago |
10-72232 10 days ago |
12-82694 12 days |
29257 |
harahu author:harahu |
doc: attach "pre", "pseudo", "semi" and "sub" as a prefixes where they are now free-standing |
These are all merely prefixes and should be attached, either in closed form or by hyphen, to some other construct.
---
[](https://gitpod.io/from-referrer/)
|
t-meta |
50/50 |
Mathlib/Algebra/Star/NonUnitalSubsemiring.lean,Mathlib/Analysis/Matrix.lean,Mathlib/Analysis/Normed/Field/WithAbs.lean,Mathlib/Analysis/Normed/Group/BallSphere.lean,Mathlib/Analysis/Normed/Module/Basic.lean,Mathlib/Lean/Meta/KAbstractPositions.lean,Mathlib/Lean/Meta/RefinedDiscrTree/Initialize.lean,Mathlib/MeasureTheory/Measure/Regular.lean,Mathlib/Probability/Martingale/BorelCantelli.lean,Mathlib/Topology/EMetricSpace/Basic.lean,Mathlib/Topology/EMetricSpace/Defs.lean,Mathlib/Topology/MetricSpace/Bounded.lean,Mathlib/Topology/MetricSpace/Gluing.lean,Mathlib/Topology/MetricSpace/IsometricSMul.lean,Mathlib/Topology/MetricSpace/ProperSpace.lean,Mathlib/Topology/MetricSpace/Pseudo/Defs.lean,Mathlib/Topology/MetricSpace/ThickenedIndicator.lean,Mathlib/Topology/MetricSpace/Thickening.lean,Mathlib/Topology/Metrizable/Basic.lean,Mathlib/Topology/Metrizable/Uniformity.lean,scripts/autolabel.lean |
21 |
1 |
['euprunin', 'github-actions'] |
JovanGerb assignee:JovanGerb |
3-34894 3 days ago |
10-57270 10 days ago |
10-57313 10 days |
29488 |
Timeroot author:Timeroot |
feat: 'said' tactic |
Functionally similar to `says`, but explicitly not for checking output or even saying there ever was output. `X said Y` just means that `X` was part of the process for (a human, or machine, or both) to generate `Y`.
Based on this [#mathlib4 > noisy simp says in CI @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/noisy.20simp.20says.20in.20CI/near/538443152) Zulip discussion
---
[](https://gitpod.io/from-referrer/)
|
|
40/0 |
Mathlib/Tactic/Linter/UnusedTactic.lean,Mathlib/Tactic/Linter/UnusedTacticExtension.lean,Mathlib/Tactic/Says.lean,MathlibTest/says.lean |
4 |
1 |
['github-actions'] |
nobody |
3-26379 3 days ago |
3-26455 3 days ago |
3-26436 3 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$ |
467/3 |
Mathlib.lean,Mathlib/Algebra/Polynomial/CoeffList.lean,Mathlib/Algebra/Polynomial/Degree/Operations.lean,Mathlib/Algebra/Polynomial/EraseLead.lean,Mathlib/Algebra/Polynomial/RuleOfSigns.lean,Mathlib/Data/Sign/Defs.lean |
6 |
27 |
['Ruben-VandeVelde', 'Timeroot', 'adomani', 'chrisflav', 'github-actions'] |
adomani assignee:adomani |
3-25645 3 days ago |
81-27628 2 months ago |
81-27669 81 days |
27262 |
Timeroot author:Timeroot |
feat(Tactic/Bound): bound? for proof scripts |
---
[](https://gitpod.io/from-referrer/)
|
t-meta |
51/40 |
Mathlib/Combinatorics/SimpleGraph/Regularity/Bound.lean,Mathlib/Combinatorics/SimpleGraph/Regularity/Lemma.lean,Mathlib/NumberTheory/Padics/Hensel.lean,Mathlib/Tactic/Bound.lean |
4 |
3 |
['JovanGerb', 'Timeroot', 'github-actions'] |
nobody |
3-21667 3 days ago |
56-55863 1 month ago |
56-55903 56 days |
29092 |
zhuyizheng author:zhuyizheng |
feat(MeasureTheory): add absolutely continuous functions, FTC and integration by parts |
Add the ε-δ definition of absolutely continuous functions on a closed interval in ℝ. Prove Fundamental Theorem of Calculus and integration by parts for absolutely continuous functions.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-measure-probability
awaiting-author
|
1376/0 |
Mathlib.lean,Mathlib/Analysis/Calculus/Deriv/Slope.lean,Mathlib/MeasureTheory/Function/AbsolutelyContinuous.lean,Mathlib/MeasureTheory/Integral/IntervalIntegral/AbsContFunc.lean,Mathlib/MeasureTheory/Integral/IntervalIntegral/DerivIntegrable.lean,Mathlib/MeasureTheory/Integral/IntervalIntegral/LebesgueDifferetiationThm.lean,Mathlib/Topology/EMetricSpace/BoundedVariation.lean |
7 |
4 |
['Ruben-VandeVelde', 'github-actions', 'grunweg'] |
nobody |
3-19205 3 days ago |
15-3889 15 days ago |
0-24361 6 hours |
29491 |
bwangpj author:bwangpj |
feat: closed point of scheme gives maximal ideal in affine open |
If a point `x` is a closed point in a scheme `X`, then its corresponding prime ideal in an affine open, `primeIdealOf x`, is maximal.
The converse is not true in general, but is true for schemes locally of finite type over a field.
---
[](https://gitpod.io/from-referrer/)
|
t-algebraic-geometry |
13/0 |
Mathlib/AlgebraicGeometry/AffineScheme.lean |
1 |
1 |
['github-actions'] |
nobody |
3-16643 3 days ago |
3-17227 3 days ago |
3-17264 3 days |
29464 |
harahu author:harahu |
doc(AkraBazzi): corrections to docs by way of LLM |
Changes are due to Junie Pro and Codex, both ChatGPT-based agents, hence warrants somewhat careful review.
I've tried to review these changes myself, but my limited lean experience is felt as a limiting factor.
Changes include:
- Fixing typos, spelling and grammar
- Changing some docstring code to LaTex math, where that seemed to be the intention
- Move some descriptions between files, in cases where definitions were promised in files they weren't defined
- Fix inconsistencies between docstrings and code (these need special review attention)
[Zulip discussion](https://leanprover.zulipchat.com/#narrow/channel/144837-PR-reviews/topic/.23.2029464.20corrections.20to.20docs.20by.20way.20of.20LLM/with/538427193)
---
[](https://gitpod.io/from-referrer/)
|
t-computability
awaiting-author
|
87/92 |
Mathlib/Computability/AkraBazzi/AkraBazzi.lean,Mathlib/Computability/AkraBazzi/GrowsPolynomially.lean,Mathlib/Computability/AkraBazzi/SumTransform.lean |
3 |
21 |
['chrisflav', 'github-actions', 'grunweg', 'harahu', 'mathlib4-merge-conflict-bot'] |
nobody |
3-11192 3 days ago |
3-11212 3 days ago |
0-6688 1 hour |
28682 |
Thmoas-Guan author:Thmoas-Guan |
feat(RingTheory): definition of regular local ring |
In this PR, we give the definition of regular local ring.
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
awaiting-author
|
117/0 |
Mathlib.lean,Mathlib/RingTheory/RegularLocalRing/Defs.lean |
2 |
34 |
['Thmoas-Guan', 'chrisflav', 'github-actions', 'mbkybky'] |
chrisflav assignee:chrisflav |
3-11092 3 days ago |
22-17715 22 days ago |
1-63449 1 day |
29479 |
harahu author:harahu |
doc: move docstring references to definitions to correct locations |
This addresses some instances of docstrings referring to results that have been moved away form their prior locations.
---
[](https://gitpod.io/from-referrer/)
|
t-computability |
14/20 |
Mathlib/Computability/AkraBazzi/AkraBazzi.lean,Mathlib/Computability/AkraBazzi/GrowsPolynomially.lean,Mathlib/Computability/AkraBazzi/SumTransform.lean |
3 |
4 |
['github-actions', 'harahu', 'mathlib4-merge-conflict-bot'] |
nobody |
3-9924 3 days ago |
3-11359 3 days ago |
3-51981 3 days |
29471 |
harahu author:harahu |
doc: use em dash instead of hyphen in Akra-Bazzi |
When joining two names, like is done here, the em dash is usually preferred over a regular hyphen.
This also aligns the naming in mathlib with that of [Wikipedia](https://en.wikipedia.org/wiki/Akra%E2%80%93Bazzi_method).
Some concern was raised [on Zulip](https://leanprover.zulipchat.com/#narrow/channel/144837-PR-reviews/topic/.23.2029464.20corrections.20to.20docs.20by.20way.20of.20LLM/near/538466767) regarding what this implies for code searches using `grep` and similar tools. Consequently, tags have been added to make sure searches using the regular hyphen will still hit the relevant files.
---
[](https://gitpod.io/from-referrer/)
|
t-computability |
29/22 |
Mathlib/Computability/AkraBazzi/AkraBazzi.lean,Mathlib/Computability/AkraBazzi/GrowsPolynomially.lean,Mathlib/Computability/AkraBazzi/SumTransform.lean |
3 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
3-9685 3 days ago |
3-11278 3 days ago |
3-65014 3 days |
29273 |
kim-em author:kim-em |
chore: add test for grind panic |
---
We can't yet merge this, as `grind` panics until we reach `v4.24.0`. |
|
65/0 |
MathlibTest/grind/panic.lean |
1 |
1 |
['github-actions'] |
nobody |
3-9107 3 days ago |
10-39311 10 days ago |
10-39292 10 days |
27841 |
CBirkbeck author:CBirkbeck |
feat(Topology/Algebra/InfiniteSum/NatInt): add more pnat tsum lemmas |
---
[](https://gitpod.io/from-referrer/)
|
t-topology |
32/7 |
Mathlib/Analysis/SpecialFunctions/Trigonometric/Cotangent.lean,Mathlib/Topology/Algebra/InfiniteSum/Basic.lean,Mathlib/Topology/Algebra/InfiniteSum/NatInt.lean |
3 |
8 |
['CBirkbeck', 'github-actions', 'loefflerd'] |
nobody |
3-5183 3 days ago |
4-59370 4 days ago |
4-60648 4 days |
28599 |
Thmoas-Guan author:Thmoas-Guan |
feat(RingTheory) : polynomial over CM ring is CM |
polynomial over Cohen Macaulay ring is Cohen Macaulay
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
large-import
|
2421/40 |
Mathlib.lean,Mathlib/Algebra/Category/Grp/Preadditive.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/LinearAlgebra/Quotient/Basic.lean,Mathlib/RingTheory/CohenMacaulay/Basic.lean,Mathlib/RingTheory/CohenMacaulay/Polynomial.lean,Mathlib/RingTheory/Ideal/AssociatedPrime/Localization.lean,Mathlib/RingTheory/Ideal/MinimalPrime/Localization.lean,Mathlib/RingTheory/Jacobson/Ideal.lean,Mathlib/RingTheory/KrullDimension/Module.lean,Mathlib/RingTheory/KrullDimension/Regular.lean,Mathlib/RingTheory/LocalRing/MaximalIdeal/Basic.lean,Mathlib/RingTheory/Nakayama.lean,Mathlib/RingTheory/Regular/Category.lean,Mathlib/RingTheory/Regular/Depth.lean,Mathlib/RingTheory/Regular/Ischebeck.lean,Mathlib/RingTheory/Support.lean |
17 |
n/a |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
3-4968 3 days ago |
unknown |
unknown |
27702 |
FLDutchmann author:FLDutchmann |
feat(NumberTheory/SelbergSieve): define Lambda-squared sieves and prove important properties |
This PR continues the work from #22052.
Original PR: https://github.com/leanprover-community/mathlib4/pull/22052
- [ ] depends on: #27820
|
t-number-theory |
199/0 |
Mathlib/NumberTheory/SelbergSieve.lean |
1 |
6 |
['FLDutchmann', 'bryangingechen', 'github-actions', 'jcommelin', 'mathlib-bors', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
3-2963 3 days ago |
3-3622 3 days ago |
3-4681 3 days |
28124 |
kckennylau author:kckennylau |
feat(Tactic): Call an arbitrary Simproc |
In the current framework, `Simproc`s are declared by name, and can only be referred to by name. For example, [Nat.divisors_ofNat](https://leanprover-community.github.io/mathlib4_docs/Mathlib/Tactic/Simproc/Divisors.html#Nat.divisors_ofNat) is declared as:
```lean
dsimproc_decl Nat.divisors_ofNat (Nat.divisors _) := fun e => do
```
This declaration syntax does not allow for a `Simproc` to depend on any arguments, and even if one constructed a `Simproc` that depends on e.g. a natural number, such as `foo : ℕ → Simproc`, one still cannot call it using the syntax `by simp [foo 37]`.
Therefore, this new function aims to solve this problem, by allowing an arbitrary `Simproc` to be executed, using the newly defined function `Lean.Meta.Simp.Simproc.apply (s : Simproc) : TacticM Unit`.
---
[](https://gitpod.io/from-referrer/)
|
t-meta |
79/0 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Simproc/Apply.lean,MathlibTest/Simproc/Apply.lean |
4 |
27 |
['JovanGerb', 'b-mehta', 'eric-wieser', 'github-actions', 'hrmacbeth', 'kckennylau'] |
JovanGerb assignee:JovanGerb |
3-1338 3 days ago |
8-59299 8 days ago |
26-28963 26 days |
29486 |
kim-em author:kim-em |
chore: scope an expensive `IsDomain`->`IsAddTorsionFree` instance |
Unfortunately this instance significantly affects (10%) the run time of
```
import Mathlib
variable {K : Type*} [Field K]
example : Lean.Grind.NoNatZeroDivisors K := inferInstance
```
which is on the critical path for `grind`. It seems okay to scope it? It is only used once, in a file with explicit `IsDomain` variables. |
t-algebra label:t-algebra$ |
12/3 |
Mathlib/Algebra/Ring/Torsion.lean,Mathlib/LinearAlgebra/RootSystem/Finite/Lemmas.lean,MathlibTest/slow_instances.lean |
3 |
4 |
['github-actions', 'kbuzzard', 'leanprover-bot'] |
nobody |
3-1045 3 days ago |
3-33057 3 days ago |
3-33098 3 days |
28780 |
gaetanserre author:gaetanserre |
feat(Analysis/SpecialFunctions): add the sigmoid function |
Add the Sigmoid from `ℝ` to `ℝ` and show some analytical properties. Then, add `sigmoid_ord_embedding`, the Sigmoid function seen as an `OrderEmbedding` from `ℝ` to `I`. Show that it is a `MeasurableEmbedding` and that we could use it to construct a `MeasurableEmbedding` from any `StandardBorelSpace` to `I`.
---
[](https://gitpod.io/from-referrer/)
|
t-analysis |
292/0 |
Mathlib.lean,Mathlib/Analysis/SpecialFunctions/Sigmoid.lean,Mathlib/Data/Set/Operations.lean |
3 |
66 |
['gaetanserre', 'github-actions', 'j-loreaux', 'themathqueen'] |
j-loreaux assignee:j-loreaux |
2-82063 2 days ago |
2-82063 2 days ago |
18-18624 18 days |
27304 |
jano-wol author:jano-wol |
feat: invariant dual submodules define Lie ideals |
Invariant dual submodules define Lie ideals
---
PR shows that Invariant dual submodules define Lie ideals.
This work is part of the framework: https://github.com/orgs/leanprover-community/projects/17
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
358/0 |
Mathlib.lean,Mathlib/Algebra/Lie/Weights/InvariantSubmoduleLieIdeal.lean,Mathlib/Algebra/Lie/Weights/Killing.lean,Mathlib/Algebra/Lie/Weights/RootSystem.lean |
4 |
1 |
['github-actions'] |
ocfnash assignee:ocfnash |
2-80304 2 days ago |
54-82492 1 month ago |
54-82535 54 days |
28789 |
yury-harmonic author:yury-harmonic |
feat(ArithmeticFunction): lemmas about positivity |
Add lemmas like `σ k n = 0 ↔ n = 0`.
Also add `positivity` extensions for `zeta` and `sigma`.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-number-theory
t-meta
awaiting-author
|
59/0 |
Mathlib/NumberTheory/ArithmeticFunction.lean,MathlibTest/positivity.lean |
2 |
7 |
['Ruben-VandeVelde', 'github-actions', 'grunweg', 'mathlib4-merge-conflict-bot', 'yury-harmonic'] |
nobody |
2-78070 2 days ago |
2-78070 2 days ago |
17-48478 17 days |
29253 |
FernandoChu author:FernandoChu |
feat(CategoryTheory): (Co)limits in preorders |
Characterize (co)limits in preorders as glbs/lubs, plus some other instances. |
new-contributor
t-category-theory
|
152/13 |
Mathlib/CategoryTheory/Discrete/Basic.lean,Mathlib/CategoryTheory/Limits/Preorder.lean,Mathlib/CategoryTheory/Limits/Shapes/BinaryProducts.lean |
3 |
7 |
['FernandoChu', 'github-actions', 'joelriou'] |
joelriou assignee:joelriou |
2-78055 2 days ago |
9-81712 9 days ago |
10-45199 10 days |
29219 |
euprunin author:euprunin |
chore: remove redundant `obtain` invocations |
---
[](https://gitpod.io/from-referrer/)
|
maintainer-merge
t-algebra
label:t-algebra$ |
0/10 |
Mathlib/Algebra/ContinuedFractions/ConvergentsEquiv.lean,Mathlib/Algebra/Homology/HomotopyCategory/Pretriangulated.lean,Mathlib/Algebra/Lie/Weights/Cartan.lean,Mathlib/Algebra/Module/PID.lean,Mathlib/Algebra/Order/Ring/Unbundled/Basic.lean,Mathlib/Algebra/Polynomial/Monic.lean |
6 |
6 |
['github-actions', 'grunweg', 'leanprover-bot', 'leanprover-community-mathlib4-bot'] |
nobody |
2-78005 2 days ago |
2-78005 2 days ago |
11-56342 11 days |
29115 |
CBirkbeck author:CBirkbeck |
feat: develop some more limUnder api |
We add results about how the `limUndet atTop` function behaves under addition, multiplication, etc. This is useful for defining the Eisensten series E2. See #28733
---
[](https://gitpod.io/from-referrer/)
|
t-topology |
105/0 |
Mathlib.lean,Mathlib/Topology/UniformSpace/LimUnder.lean |
2 |
10 |
['CBirkbeck', 'github-actions', 'j-loreaux', 'loefflerd', 'mathlib4-merge-conflict-bot', 'plp127'] |
j-loreaux assignee:j-loreaux |
2-75084 2 days ago |
12-2123 12 days ago* |
14-60582 14 days* |
29506 |
Vierkantor author:Vierkantor |
feat(CI): `nightly-testing` regression report |
This PR adds a workflow that builds the `nightly-testing-green` branch with extra linting options enabled, and reports the results on Zulip. We currently can use this to catch places where `grind` doesn't solve goals that `linarith`/`omega`/`ring` can solve.
Example output to Zulip:
> Mathlib's [nightly-testing branch](https://github.com/leanprover-community/mathlib4-nightly-testing/tree/nightly-testing) ([0f4ee783b5dac29751bce6be710a445e89159a69](https://github.com/Vierkantor/mathlib4/commit/0f4ee783b5dac29751bce6be710a445e89159a69)) regression run [completed](https://github.com/Vierkantor/mathlib4/actions/runs/17583902916).
> Warnings: 283
>
> | | Warning description |
> | ---: | --- |
> | 235 | `grind` failed where `linarith` succeeded. |
> | 45 | `grind` failed where `ring` succeeded. |
> | 2 | original tactic 'linarith' failed: linarith failed to find a contradiction |
> | 1 | original tactic 'linarith [(Nat.find_spec h_exist).1]' failed: failed to synthesize |
---
[](https://gitpod.io/from-referrer/)
|
CI |
186/6 |
.github/workflows/nightly-regression-report.yml,Mathlib/Tactic/TacticAnalysis/Declarations.lean,scripts/zulip_build_report.sh |
3 |
1 |
['github-actions'] |
nobody |
2-70628 2 days ago |
2-70693 2 days ago |
2-70675 2 days |
27306 |
xyzw12345 author:xyzw12345 |
feat: `lie_ring` tactic and `LieReduce` command |
This PR continues the work from #22196.
Original PR: https://github.com/leanprover-community/mathlib4/pull/22196 |
t-meta |
783/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 |
6 |
['JovanGerb', 'github-actions', 'xyzw12345'] |
JovanGerb assignee:JovanGerb |
2-70451 2 days ago |
4-25508 4 days ago |
51-78990 51 days |
29045 |
grunweg author:grunweg |
chore: remove the `field_simps` simp set |
This was used for the field_simp tactic before its recent rewrite. Its uses in mathlib were removed in #28918.
---
- [x] depends on: #28918
[](https://gitpod.io/from-referrer/)
|
maintainer-merge |
31/82 |
Mathlib/Algebra/CharP/MixedCharZero.lean,Mathlib/Algebra/Field/Basic.lean,Mathlib/Algebra/Group/Basic.lean,Mathlib/Algebra/Group/Defs.lean,Mathlib/Algebra/Group/Units/Basic.lean,Mathlib/Algebra/Group/Units/Defs.lean,Mathlib/Algebra/GroupWithZero/Basic.lean,Mathlib/Algebra/GroupWithZero/Units/Basic.lean,Mathlib/Algebra/NeZero.lean,Mathlib/Algebra/Order/Field/Basic.lean,Mathlib/Algebra/Ring/Basic.lean,Mathlib/Algebra/Ring/Units.lean,Mathlib/Analysis/Complex/Trigonometric.lean,Mathlib/Analysis/InnerProductSpace/Basic.lean,Mathlib/Analysis/MeanInequalitiesPow.lean,Mathlib/Analysis/Normed/Unbundled/SeminormFromBounded.lean,Mathlib/Analysis/Normed/Unbundled/SeminormFromConst.lean,Mathlib/Analysis/Normed/Unbundled/SmoothingSeminorm.lean,Mathlib/Combinatorics/SetFamily/AhlswedeZhang.lean,Mathlib/Combinatorics/SimpleGraph/Density.lean,Mathlib/MeasureTheory/Measure/Haar/Basic.lean,Mathlib/Tactic/Attr/Register.lean |
22 |
7 |
['Ruben-VandeVelde', 'bryangingechen', 'github-actions', 'grunweg', 'mathlib4-dependent-issues-bot'] |
nobody |
2-67785 2 days ago |
6-53156 6 days ago |
15-52021 15 days |
29500 |
vihdzp author:vihdzp |
feat: `WellFoundedLT (LowerSet α)` |
We prove that `LowerSet α` is well-founded when `α` is a WQO.
---
This result is used in the CGT repository to construct the poset game!
[](https://gitpod.io/from-referrer/)
|
t-order |
31/0 |
Mathlib.lean,Mathlib/Order/UpperLower/WellFounded.lean |
2 |
2 |
['github-actions', 'plp127'] |
nobody |
2-67665 2 days ago |
2-77630 2 days ago |
2-77673 2 days |
29504 |
zhuyizheng author:zhuyizheng |
feat(MeasureTheory): add absolutely continuous functions |
Add absolutely continuous functions. Part of originally planned #29092.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-measure-probability
|
375/0 |
Mathlib.lean,Mathlib/MeasureTheory/Function/AbsolutelyContinuous.lean,Mathlib/Topology/EMetricSpace/BoundedVariation.lean |
3 |
1 |
['github-actions'] |
nobody |
2-65847 2 days ago |
2-65847 2 days ago |
2-72687 2 days |
29113 |
scholzhannah author:scholzhannah |
chore: rename PartialHomeomorph to OpenPartialHomeomorph |
This PR renames `PartialHomeomorph` to `OpenPartialHomeomorph` as discussed in [#mathlib4 > Generalizing `PartialHomeomorph`?](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Generalizing.20.60PartialHomeomorph.60.3F). This is the first step towards generalizing `PartialHomeomorph` to allow arbitrary sources and targets.
---
This is the first time that I am doing this type of renaming. I tried to do everything well but I am not sure that I did it how it is supposed to be done.
[](https://gitpod.io/from-referrer/)
|
file-removed |
1257/1021 |
Mathlib.lean,Mathlib/Analysis/Analytic/Inverse.lean,Mathlib/Analysis/Asymptotics/Defs.lean,Mathlib/Analysis/Asymptotics/Lemmas.lean,Mathlib/Analysis/Calculus/ContDiff/Operations.lean,Mathlib/Analysis/Calculus/Deriv/Inverse.lean,Mathlib/Analysis/Calculus/FDeriv/Analytic.lean,Mathlib/Analysis/Calculus/FDeriv/Equiv.lean,Mathlib/Analysis/Calculus/Implicit.lean,Mathlib/Analysis/Calculus/InverseFunctionTheorem/ApproximatesLinearOn.lean,Mathlib/Analysis/Calculus/InverseFunctionTheorem/ContDiff.lean,Mathlib/Analysis/Calculus/InverseFunctionTheorem/FDeriv.lean,Mathlib/Analysis/Complex/Tietze.lean,Mathlib/Analysis/Complex/UpperHalfPlane/Topology.lean,Mathlib/Analysis/InnerProductSpace/Calculus.lean,Mathlib/Analysis/Normed/Module/Ball/Homeomorph.lean,Mathlib/Analysis/SpecialFunctions/Arsinh.lean,Mathlib/Analysis/SpecialFunctions/Complex/LogDeriv.lean,Mathlib/Analysis/SpecialFunctions/Log/Basic.lean,Mathlib/Analysis/SpecialFunctions/PolarCoord.lean,Mathlib/Analysis/SpecialFunctions/Sqrt.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Arctan.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Inverse.lean,Mathlib/Deprecated/AnalyticManifold.lean,Mathlib/Geometry/Manifold/ChartedSpace.lean,Mathlib/Geometry/Manifold/ConformalGroupoid.lean,Mathlib/Geometry/Manifold/ContMDiff/Atlas.lean,Mathlib/Geometry/Manifold/ContMDiff/Basic.lean,Mathlib/Geometry/Manifold/ContMDiff/Defs.lean,Mathlib/Geometry/Manifold/ContMDiffMFDeriv.lean,Mathlib/Geometry/Manifold/Diffeomorph.lean,Mathlib/Geometry/Manifold/Instances/Icc.lean,Mathlib/Geometry/Manifold/Instances/Real.lean,Mathlib/Geometry/Manifold/Instances/Sphere.lean,Mathlib/Geometry/Manifold/IsManifold/Basic.lean,Mathlib/Geometry/Manifold/IsManifold/ExtChartAt.lean,Mathlib/Geometry/Manifold/IsManifold/InteriorBoundary.lean,Mathlib/Geometry/Manifold/LocalDiffeomorph.lean,Mathlib/Geometry/Manifold/LocalInvariantProperties.lean,Mathlib/Geometry/Manifold/MFDeriv/Atlas.lean,Mathlib/Geometry/Manifold/MFDeriv/Basic.lean,Mathlib/Geometry/Manifold/MFDeriv/Defs.lean,Mathlib/Geometry/Manifold/MFDeriv/Tangent.lean,Mathlib/Geometry/Manifold/MFDeriv/UniqueDifferential.lean,Mathlib/Geometry/Manifold/PartitionOfUnity.lean,Mathlib/Geometry/Manifold/VectorBundle/Basic.lean,Mathlib/Geometry/Manifold/VectorBundle/FiberwiseLinear.lean,Mathlib/Geometry/Manifold/VectorBundle/Hom.lean,Mathlib/Geometry/Manifold/VectorBundle/MDifferentiable.lean,Mathlib/Geometry/Manifold/VectorBundle/Tangent.lean,Mathlib/Logic/Equiv/PartialEquiv.lean,Mathlib/MeasureTheory/Function/Jacobian.lean,Mathlib/NumberTheory/ModularForms/EisensteinSeries/UniformConvergence.lean,Mathlib/NumberTheory/NumberField/CanonicalEmbedding/NormLeOne.lean,Mathlib/NumberTheory/NumberField/CanonicalEmbedding/PolarCoord.lean,Mathlib/Topology/Covering.lean,Mathlib/Topology/FiberBundle/Basic.lean,Mathlib/Topology/FiberBundle/Constructions.lean,Mathlib/Topology/FiberBundle/Trivialization.lean,Mathlib/Topology/Instances/AddCircle/Defs.lean,Mathlib/Topology/IsLocalHomeomorph.lean,Mathlib/Topology/OpenPartialHomeomorph.lean,Mathlib/Topology/VectorBundle/Basic.lean,MathlibTest/MfldSetTac.lean |
64 |
12 |
['github-actions', 'grunweg', 'mathlib4-merge-conflict-bot'] |
nobody |
2-63690 2 days ago |
2-63710 2 days ago |
11-20484 11 days |
29156 |
harahu author:harahu |
doc: treat "non" as a prefix where it appears as a free-standing word |
In English, "non" is merely a prefix, not a word in itself. Hence, it should always be attached to another word, either directly or by hyphen.
This PR attaches the prefix "non" to whatever it is prefixing in the cases where it currently appears as a free-standing word.
There's a couple of tricky cases in the PR that needs some extra attention. I will call these out by review comments.
---
[](https://gitpod.io/from-referrer/)
|
|
89/89 |
Mathlib/Algebra/Group/Defs.lean,Mathlib/Algebra/Order/Hom/Basic.lean,Mathlib/Algebra/Order/Sub/Basic.lean,Mathlib/Algebra/Ring/BooleanRing.lean,Mathlib/Algebra/Ring/CentroidHom.lean,Mathlib/Algebra/Ring/Defs.lean,Mathlib/Algebra/Star/CentroidHom.lean,Mathlib/AlgebraicTopology/DoldKan/Degeneracies.lean,Mathlib/Analysis/Complex/Arg.lean,Mathlib/Analysis/Complex/Polynomial/Basic.lean,Mathlib/Analysis/InnerProductSpace/Basic.lean,Mathlib/Analysis/Normed/Group/Basic.lean,Mathlib/Analysis/Normed/Unbundled/RingSeminorm.lean,Mathlib/Analysis/SpecialFunctions/NonIntegrable.lean,Mathlib/CategoryTheory/Closed/Ideal.lean,Mathlib/CategoryTheory/Filtered/Basic.lean,Mathlib/CategoryTheory/Monoidal/Category.lean,Mathlib/CategoryTheory/Monoidal/Mod_.lean,Mathlib/CategoryTheory/SmallObject/Iteration/Basic.lean,Mathlib/Combinatorics/Additive/AP/Three/Defs.lean,Mathlib/Combinatorics/SimpleGraph/Regularity/Uniform.lean,Mathlib/Data/Finsupp/Weight.lean,Mathlib/FieldTheory/Finite/GaloisField.lean,Mathlib/FieldTheory/RatFunc/Basic.lean,Mathlib/GroupTheory/Perm/Cycle/Basic.lean,Mathlib/GroupTheory/Perm/Sign.lean,Mathlib/Order/BooleanAlgebra/Basic.lean,Mathlib/Order/CompleteBooleanAlgebra.lean,Mathlib/Order/Disjoint.lean,Mathlib/Order/GaloisConnection/Basic.lean,Mathlib/Order/Interval/Finset/Defs.lean,Mathlib/Order/Partition/Finpartition.lean,Mathlib/Order/SuccPred/Archimedean.lean,Mathlib/Order/SuccPred/Basic.lean,Mathlib/Order/TransfiniteIteration.lean,Mathlib/Probability/ProductMeasure.lean,Mathlib/RingTheory/KrullDimension/NonZeroDivisors.lean,Mathlib/RingTheory/LocalRing/MaximalIdeal/Defs.lean,Mathlib/RingTheory/MvPolynomial/MonomialOrder.lean,Mathlib/RingTheory/MvPolynomial/WeightedHomogeneous.lean,Mathlib/RingTheory/MvPowerSeries/Order.lean,Mathlib/RingTheory/OrderOfVanishing.lean,Mathlib/RingTheory/Polynomial/Eisenstein/Criterion.lean,Mathlib/RingTheory/Regular/IsSMulRegular.lean,Mathlib/SetTheory/Ordinal/Basic.lean,Mathlib/Topology/Algebra/Nonarchimedean/Bases.lean,Mathlib/Topology/Algebra/Valued/ValuationTopology.lean,Mathlib/Topology/Baire/BaireMeasurable.lean,Mathlib/Topology/Connected/LocallyConnected.lean,Mathlib/Topology/ContinuousMap/StoneWeierstrass.lean,Mathlib/Topology/Sets/Compacts.lean |
51 |
70 |
['github-actions', 'grunweg', 'harahu', 'mathlib4-merge-conflict-bot'] |
nobody |
2-60996 2 days ago |
2-61018 2 days ago |
10-76931 10 days |
29511 |
luigi-massacci author:luigi-massacci |
feat: integrating wrt a finite measure as a continuous linear map on bounded continuous functions |
Add a definition `integralFiniteMeasure` of type `ContinuousLinearMap` packaging the integral of a bounded continuous function by a finite measure.
---
[](https://gitpod.io/from-referrer/)
|
maintainer-merge
t-measure-probability
|
17/0 |
Mathlib/MeasureTheory/Integral/BoundedContinuousFunction.lean |
1 |
23 |
['github-actions', 'grunweg', 'luigi-massacci'] |
nobody |
2-58639 2 days ago |
2-58640 2 days ago |
2-60785 2 days |
29514 |
grunweg author:grunweg |
More strict mode |
---
[](https://gitpod.io/from-referrer/)
|
CI
WIP
|
192/33 |
.github/build.in.yml,.github/workflows/bors.yml,.github/workflows/build.yml,.github/workflows/build_fork.yml,Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter/ValidatePRTitle.lean,lakefile.lean,scripts/README.md,scripts/check_title_labels.lean |
10 |
1 |
['github-actions'] |
nobody |
2-58100 2 days ago |
2-58167 2 days ago |
0-1 1 second |
25324 |
eric-wieser author:eric-wieser |
feat: more functorial results about DFinsupp |
We have these already for Finsupp.
The `DFinsupp` statements need some extra casts in some places.
---
- [ ] depends on: #27182
[](https://gitpod.io/from-referrer/)
[#mathlib4 > Equiv.cast for structures @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Equiv.2Ecast.20for.20structures/near/521390935)
|
t-data
t-algebra
label:t-algebra$ |
137/16 |
Mathlib/Data/DFinsupp/Defs.lean,Mathlib/LinearAlgebra/DFinsupp.lean |
2 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
2-57381 2 days ago |
2-57536 2 days ago |
2-57514 2 days |
29498 |
harahu author:harahu |
doc: improve grammar and flow in documentation |
This PR might be deemed too stylistic in nature, but I'll propose it anyhow, with the purpose of sectioning out potential for bikeshedding from #29464.
The changes are largely the work of LLM coding agents, but I have manually checked every change and have not included anything in this PR that I cannot personally stand for.
In totality, my opinion is that this PR improves the legibility, clarity and conciseness of the documentation it covers, and should be merged.
---
[](https://gitpod.io/from-referrer/)
|
maintainer-merge
t-computability
|
40/39 |
Mathlib/Computability/AkraBazzi/AkraBazzi.lean,Mathlib/Computability/AkraBazzi/GrowsPolynomially.lean,Mathlib/Computability/AkraBazzi/SumTransform.lean |
3 |
12 |
['github-actions', 'grunweg', 'harahu', 'themathqueen'] |
nobody |
2-57320 2 days ago |
2-72249 2 days ago |
2-78229 2 days |
29057 |
jeremypparker author:jeremypparker |
feat(Topology/Instances): `AddCircle.liftIoc_continuous` |
Previously `AddCircle.liftIco_continuous` existed but this equivalent result did not. In the process I prove that
`liftIoc` is equivalent to `liftIco` if the endpoint values are equal.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-topology
|
50/5 |
Mathlib/Topology/Instances/AddCircle/Defs.lean |
1 |
8 |
['Ruben-VandeVelde', 'github-actions', 'jeremypparker'] |
ADedecker assignee:ADedecker |
2-50757 2 days ago |
15-83442 15 days ago |
15-83478 15 days |
29380 |
chrisflav author:chrisflav |
feat(CategoryTheory/MorphismProperty): define `ind P` |
Given a morphism property `P`, we define a morphism property `ind P` that is satisfied for
`f : X ⟶ Y` if `Y` is a filtered colimit of `Yᵢ` and `fᵢ : X ⟶ Yᵢ` satisfy `P`.
We show that `ind` is idempotent under certain compactness assumptions.
---
- [x] depends on: #29382
[](https://gitpod.io/from-referrer/)
|
large-import
t-category-theory
|
289/0 |
Mathlib.lean,Mathlib/CategoryTheory/Limits/Presentation.lean,Mathlib/CategoryTheory/MorphismProperty/Comma.lean,Mathlib/CategoryTheory/MorphismProperty/Ind.lean,Mathlib/CategoryTheory/ObjectProperty/Ind.lean,Mathlib/CategoryTheory/Presentable/Finite.lean,Mathlib/CategoryTheory/WithTerminal/Lemmas.lean |
7 |
13 |
['chrisflav', 'github-actions', 'joelriou', 'mathlib4-dependent-issues-bot'] |
nobody |
2-50622 2 days ago |
2-50622 2 days ago |
4-255 4 days |
28395 |
joelriou author:joelriou |
feat(AlgebraicTopology/SimplicialSet): nondegenerate simplices in the standard simplex |
In this PR, we show that `d`-dimensional nondegenerate simplices in `Δ[n]` identify to `Fin (d + 1) ↪o Fin (n + 1)`.
(This PR also contains some general additional API for (non)degenerate simplices. For this reason, three definitions related to subcomplexes generated by a simplex had to be moved from `StdSimplex.lean` to `Subcomplex.lean`.)
---
- [x] depends on: #28337
[](https://gitpod.io/from-referrer/)
|
t-algebraic-topology |
248/20 |
Mathlib/AlgebraicTopology/SimplicialSet/Degenerate.lean,Mathlib/AlgebraicTopology/SimplicialSet/Simplices.lean,Mathlib/AlgebraicTopology/SimplicialSet/StdSimplex.lean,Mathlib/AlgebraicTopology/SimplicialSet/Subcomplex.lean,Mathlib/Order/Hom/Basic.lean |
5 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
2-50238 2 days ago |
2-59859 2 days ago |
2-59840 2 days |
29478 |
llllvvuu author:llllvvuu |
feat(LinearAlgebra): roots of charpoly are the eigenvalues/spectrum |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
79/10 |
Mathlib.lean,Mathlib/LinearAlgebra/Eigenspace/Charpoly.lean,Mathlib/LinearAlgebra/Eigenspace/Matrix.lean,Mathlib/LinearAlgebra/Matrix/Charpoly/Eigs.lean |
4 |
9 |
['github-actions', 'llllvvuu', 'themathqueen'] |
nobody |
2-49324 2 days ago |
3-58174 3 days ago |
3-58187 3 days |
29516 |
kckennylau author:kckennylau |
chore: Deprecate IsAdjoinRoot.subsingleton |
This PR deprecates `IsAdjoinRoot.subsingleton` in favour of the new `Algebra.subsingleton`:
```lean
theorem IsAdjoinRoot.subsingleton {R : Type u} {S : Type v} [CommRing R] [Ring S] {f : Polynomial R}
[Algebra R S] (h : IsAdjoinRoot S f) [Subsingleton R] :
Subsingleton S
theorem Algebra.subsingleton (R : Type u) (A : Type v) [CommSemiring R] [Semiring A] [Algebra R A]
[Subsingleton R] : Subsingleton A
```
---
Zulip: https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/IsAdjoinRoot.2Esubsingleton/with/538731602
[](https://gitpod.io/from-referrer/)
|
|
9/3 |
Mathlib/Algebra/Algebra/Defs.lean,Mathlib/RingTheory/IsAdjoinRoot.lean |
2 |
1 |
['github-actions'] |
nobody |
2-47494 2 days ago |
2-51255 2 days ago |
2-51236 2 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 |
7 |
['Paul-Lez', 'eric-wieser', 'github-actions', 'kckennylau'] |
nobody |
2-47109 2 days ago |
151-51434 4 months ago |
151-51479 151 days |
29405 |
pechersky author:pechersky |
feat(NumberTheory/Padic): characterization of norms of zmodRepr |
And of `p - 1`
In preparation for `p - 1` roots of unity
---
[](https://gitpod.io/from-referrer/)
Instead of using general `IsUltrametricDist` lemmas, prefer to use lower level specialized lemmas to prevent import increase |
t-number-theory |
123/0 |
Mathlib/NumberTheory/Padics/PadicIntegers.lean,Mathlib/NumberTheory/Padics/PadicNumbers.lean,Mathlib/NumberTheory/Padics/RingHoms.lean |
3 |
1 |
['github-actions'] |
nobody |
2-46946 2 days ago |
5-58397 5 days ago |
5-58385 5 days |
29403 |
pechersky author:pechersky |
feat(Data/Nat/Basic): Nat.dvd_sub_self_iff |
a lemma to deal with a trivial side case
---
[](https://gitpod.io/from-referrer/)
|
t-data
easy
|
18/0 |
Mathlib/Data/Nat/Basic.lean |
1 |
2 |
['Ruben-VandeVelde', 'github-actions'] |
nobody |
2-46933 2 days ago |
5-37249 5 days ago |
5-52063 5 days |
29416 |
pechersky author:pechersky |
feat(RingTheoryy/RootsOfUnity): of_card_le |
If the cardinality of n-th roots of unity is >= n, then `HasEnoughRootsOfUnity` the reverse direction of `natCard_rootsOfUnity`
but requires `CommRing`
Stated with an `LE` instead of `Eq` to have a weaker hypothesis
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory |
17/0 |
Mathlib/RingTheory/RootsOfUnity/EnoughRootsOfUnity.lean |
1 |
1 |
['github-actions'] |
nobody |
2-46883 2 days ago |
5-36993 5 days ago |
5-36981 5 days |
29408 |
pechersky author:pechersky |
feat(Analysis/Normed/Ultra): nonarch norm of sum over disjoint norms achieves max |
---
[](https://gitpod.io/from-referrer/)
I thought about having a `tprod` version too, but wasn't sure the best way to phrase it
|
maintainer-merge
t-analysis
|
24/0 |
Mathlib/Analysis/Normed/Group/Ultra.lean |
1 |
5 |
['github-actions', 'loefflerd'] |
nobody |
2-46849 2 days ago |
4-76226 4 days ago |
5-57569 5 days |
28349 |
kckennylau author:kckennylau |
feat(Meta): add notation for naming stacked polynomials |
This PR changes the notation for naming formal variables associated to recursive polynomial-like objects.
Registration is done only once per each polynomial-like functor.
Usage:
```lean
#register_poly_vars "[" X "]" Polynomial Polynomial.C Polynomial.X
#register_poly_vars "[" X, ... "]" MvPolynomial MvPolynomial.C MvPolynomial.X
#name_poly_vars R[a,b][C]
#name_poly_vars _[[x,y,z]]
```
`_[[x,y,z]]` allows for the hole to be substituted by any base ring, so `(x : R[[x,y,z]])` will make sense.
---
I have not mass deployed the new syntax at every possible location, I plan to do that in a future PR following this.
Zulip: [#mathlib4 > Notation for polynomial variables](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Notation.20for.20polynomial.20variables)
[](https://gitpod.io/from-referrer/)
|
t-meta |
386/57 |
Counterexamples/CliffordAlgebraNotInjective.lean,Mathlib/Algebra/MvPolynomial/Basic.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Jacobian/Basic.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Projective/Basic.lean,Mathlib/Tactic/Ring/NamePolyVars.lean,MathlibTest/NamePolyVars.lean |
6 |
19 |
['adamtopaz', 'eric-wieser', 'github-actions', 'kckennylau', 'plp127'] |
adamtopaz assignee:adamtopaz |
2-44409 2 days ago |
2-47781 2 days ago |
29-51407 29 days |
29518 |
joelriou author:joelriou |
feat(CategoryTheory): extremal epimorphisms |
An extremal epimorphism `p : X ⟶ Y` is an epimorphism which does not factor through any proper subobject of `Y`. In case the category has equalizers, we show that a morphism `p : X ⟶ Y` which does not factor through any proper subobject of `Y` is automatically an epimorphism, and also an extremal epimorphism. We also show that a strong epimorphism is an extremal epimorphism, and that both notions coincide when the category has pullbacks.
---
[](https://gitpod.io/from-referrer/)
|
t-category-theory |
75/0 |
Mathlib.lean,Mathlib/CategoryTheory/ExtremalEpi.lean |
2 |
3 |
['github-actions', 'joelriou'] |
nobody |
2-39856 2 days ago |
2-41390 2 days ago |
2-41373 2 days |
26031 |
joelriou author:joelriou |
feat(Algebra/Homology): the derived category of a linear abelian category is linear |
---
- [x] depends on: #25931
This PR continues the work from #24596.
Original PR: https://github.com/leanprover-community/mathlib4/pull/24596 |
t-category-theory |
71/0 |
Mathlib.lean,Mathlib/Algebra/Homology/DerivedCategory/Linear.lean,Mathlib/Algebra/Homology/HomotopyCategory/Shift.lean,Mathlib/Algebra/Homology/HomotopyCategory/SingleFunctors.lean |
4 |
n/a |
['AntoineChambert-Loir', 'github-actions', 'joelriou', 'mathlib4-dependent-issues-bot'] |
nobody |
2-39225 2 days ago |
unknown |
unknown |
28614 |
kckennylau author:kckennylau |
feat(CategoryTheory): The finite pretopology on a category |
We define `CategoryTheory.Pretopology.finite`, the finite pretopology on a category, which consists of presieves that contain only finitely many arrows.
---
[](https://gitpod.io/from-referrer/)
|
maintainer-merge
t-category-theory
|
131/0 |
Mathlib.lean,Mathlib/CategoryTheory/Sites/Finite.lean,Mathlib/CategoryTheory/Sites/Sieves.lean |
3 |
31 |
['chrisflav', 'github-actions', 'joelriou', 'kckennylau'] |
chrisflav assignee:chrisflav |
2-39169 2 days ago |
2-49232 2 days ago |
10-83876 10 days |
29221 |
euprunin author:euprunin |
chore: remove redundant `rintro` invocations (before `omega`) |
---
[](https://gitpod.io/from-referrer/)
|
|
0/4 |
Mathlib/Algebra/BigOperators/Intervals.lean,Mathlib/Algebra/Group/Nat/Range.lean,Mathlib/Data/List/Range.lean |
3 |
4 |
['github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot'] |
RemyDegenne assignee:RemyDegenne |
2-34909 2 days ago |
10-47446 10 days ago |
11-54540 11 days |
29239 |
harahu author:harahu |
Doc: Hyphenize compound adjectives ending in "-valued" |
---
[](https://gitpod.io/from-referrer/)
|
|
54/54 |
Mathlib/Algebra/BigOperators/Group/Finset/Basic.lean,Mathlib/AlgebraicGeometry/ProjectiveSpectrum/StructureSheaf.lean,Mathlib/AlgebraicGeometry/StructureSheaf.lean,Mathlib/Analysis/Calculus/Deriv/Comp.lean,Mathlib/Analysis/Calculus/Taylor.lean,Mathlib/Analysis/Complex/UpperHalfPlane/FunctionsBoundedAtInfty.lean,Mathlib/Analysis/MeanInequalities.lean,Mathlib/Analysis/NormedSpace/MultipliableUniformlyOn.lean,Mathlib/CategoryTheory/Functor/ReflectsIso/Basic.lean,Mathlib/CategoryTheory/Limits/Cones.lean,Mathlib/CategoryTheory/Simple.lean,Mathlib/CategoryTheory/Sites/Subsheaf.lean,Mathlib/CategoryTheory/Subpresheaf/Basic.lean,Mathlib/Data/Sigma/Basic.lean,Mathlib/FieldTheory/Relrank.lean,Mathlib/Geometry/Manifold/Riemannian/Basic.lean,Mathlib/Geometry/RingedSpace/SheafedSpace.lean,Mathlib/MeasureTheory/Constructions/BorelSpace/Real.lean,Mathlib/MeasureTheory/Function/ConditionalExpectation/Real.lean,Mathlib/MeasureTheory/VectorMeasure/Basic.lean,Mathlib/NumberTheory/Padics/PadicNumbers.lean,Mathlib/Probability/Martingale/Upcrossing.lean,Mathlib/Probability/StrongLaw.lean,Mathlib/Tactic/CategoryTheory/MonoidalComp.lean,Mathlib/Tactic/FunProp/Decl.lean,Mathlib/Tactic/Linarith/Frontend.lean,Mathlib/Topology/Algebra/InfiniteSum/ENNReal.lean,Mathlib/Topology/EMetricSpace/BoundedVariation.lean,Mathlib/Topology/Separation/CompletelyRegular.lean,Mathlib/Topology/Sheaves/CommRingCat.lean,Mathlib/Topology/Sheaves/Sheafify.lean,docs/undergrad.yaml |
32 |
2 |
['github-actions', 'harahu'] |
riccardobrasca assignee:riccardobrasca |
2-34908 2 days ago |
10-83400 10 days ago |
10-83381 10 days |
29300 |
Louddy author:Louddy |
feat: SkewPolynomial |
# Univariate skew polynomials
Skew polynomials are represented as `SkewMonoidAlgebra R (Multiplicative ℕ)`, where `R` is usually at least a Semiring.
In this file, we define `SkewPolynomial` and provide basic instances.
The point if this PR is to introduce the very most basic definitions and API.
From #23949.
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$ |
178/0 |
Mathlib.lean,Mathlib/Algebra/SkewPolynomial/Basic.lean,docs/references.bib |
3 |
1 |
['github-actions'] |
joelriou assignee:joelriou |
2-34901 2 days ago |
10-302 10 days ago |
10-332 10 days |
29315 |
kbuzzard author:kbuzzard |
chore: raise priority of `IsTopologicalSemiring.toIsModuleTopology` |
Instances of the form `SMul A B -> SMul (F A) (F B)` can be problematic for several reasons, one of them being that if `A = B` is a ring and if `F A` is also ring then this can cause a diamond with `Algebra.id`. In mathlib we attempt to coerce typeclass inference away from such problems by raising the priority of `Algebra.id` to 1100; this hack (implemented in #13032) seems to work well, indeed it seems sensible to try this instance early because it should be quick to fail and is always the right idea when it doesn't (the change also made mathlib faster and made a proof better). By the same logic it seems safe to raise the priority of `IsTopologicalSemiring.toIsModuleTopology` by the same amount; in FLT there is a mathematically natural but mathlib-problematic instance `Algebra K L -> Algebra (𝔸 K) (𝔸 L)`
and then another instance `Algebra K L -> IsModuleTopology (𝔸 K) (𝔸 L)` where `𝔸 K` is the adele ring of the number field `K`, and the change in this PR solves timeouts when `K = L`.
Zulip: [#mathlib4 > product of modules over product of rings @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/product.20of.20modules.20over.20product.20of.20rings/near/532799613)
---
[](https://gitpod.io/from-referrer/)
There are other solutions to this problem -- I am certainly not claiming that the FLT project needs this PR to be merged! We can tinker with priorities locally in FLT for example. However when I noticed that `Algebra.id` had a raised priority in mathlib I realised that mathlib might be amenable to this further ~~hack~~change.
|
t-topology |
6/1 |
Mathlib/Topology/Algebra/Module/ModuleTopology.lean |
1 |
4 |
['github-actions', 'kbuzzard', 'leanprover-bot'] |
j-loreaux assignee:j-loreaux |
2-34900 2 days ago |
9-77045 9 days ago |
9-77086 9 days |
29302 |
harahu author:harahu |
doc: hyphenate attributive compound adjectives starting with "upper" or "lower" |
Compound adjectives that are attributive (coming before their noun) should almost always be hyphenated in English.
This PR covers such adjectives that are starting with "upper" or "lower".
---
[](https://gitpod.io/from-referrer/)
|
|
53/53 |
Mathlib/Analysis/LocallyConvex/Barrelled.lean,Mathlib/MeasureTheory/Integral/Bochner/VitaliCaratheodory.lean,Mathlib/Order/ModularLattice.lean,Mathlib/Topology/Semicontinuous.lean |
4 |
1 |
['github-actions'] |
EtienneC30 assignee:EtienneC30 |
2-34900 2 days ago |
10-2767 10 days ago |
10-2748 10 days |
29318 |
FernandoChu author:FernandoChu |
feat(CategoryTheory): (Co)limits in skeletons |
As [suggested in the zulip](https://leanprover.zulipchat.com/#narrow/channel/217875-Is-there-code-for-X.3F/topic/Transporting.20properties.20along.20an.20equivalence.20of.20cats/with/533308058), I add here some instances for (co)limits in the skeletons. This is useful, e.g., for showing that `Subobject X` has arbitrary suprema/infima under some conditions in the underlying category. |
new-contributor
t-category-theory
|
79/3 |
Mathlib.lean,Mathlib/CategoryTheory/Limits/Skeleton.lean,Mathlib/CategoryTheory/Skeletal.lean |
3 |
1 |
['github-actions'] |
robin-carlier assignee:robin-carlier |
2-34899 2 days ago |
9-72574 9 days ago |
9-72611 9 days |
29497 |
xyzw12345 author:xyzw12345 |
feat(Counterexamples): A ring such that dim A = 1 but dim A[x] = 3 |
In this PR, we constructed an example of a commutative ring `A` that satisfies `ringKrullDim A = 1` but `ringKrullDim A[X] = 3`, following the construction of
https://math.stackexchange.com/questions/1267419/examples-of-rings-whose-polynomial-rings-have-large-dimension
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
162/0 |
Counterexamples.lean,Counterexamples/DimensionPolynomial.lean,Mathlib/Algebra/Ring/Subring/Basic.lean,Mathlib/FieldTheory/RatFunc/AsPolynomial.lean,Mathlib/RingTheory/LocalRing/MaximalIdeal/Basic.lean |
5 |
11 |
['github-actions', 'kbuzzard', 'kckennylau', 'xyzw12345'] |
nobody |
2-34037 2 days ago |
3-6115 3 days ago |
3-6143 3 days |
29527 |
kim-em author:kim-em |
feat: script for checking Github URLs |
This adds scripts/check_github_urls.py, which checks for links for closed github issues/prs, and shows the context at the link.
Of course, many links are to closed pull requests because the discussion there provides useful context. Not sure how to best filter results. |
CI
WIP
|
475/0 |
scripts/README.md,scripts/check_github_urls.py |
2 |
2 |
['github-actions', 'kim-em'] |
nobody |
2-32442 2 days ago |
2-33122 2 days ago |
0-1 1 second |
29526 |
llllvvuu author:llllvvuu |
feat: `Multiset.map f` identifies `f` up to permutation |
Example use case: Reason about `Matrix.IsHermitian.eigenvalues`, which is `Fintype`-indexed, via `Matrix.charpoly.roots` which is a `Multiset`.
---
[](https://gitpod.io/from-referrer/)
|
t-data |
29/0 |
Mathlib/Data/Multiset/Fintype.lean |
1 |
1 |
['github-actions'] |
nobody |
2-30863 2 days ago |
2-33318 2 days ago |
2-33316 2 days |
29532 |
Aaron1011 author:Aaron1011 |
feat: add group/field versions of Filter.map_*_atTop_eq_nat |
Add Filter.map_add_atTop_eq, Filter.map_sub_atTop_eq, and Filter.map_div_atTop_eq, which correspond to
Filter.map_add_atTop_eq_nat, Filter.map_sub_atTop_eq_nat, and Filter.map_div_atTop_eq_nat respectively.
These theorems apply to ordered groups/fields
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-order
|
14/0 |
Mathlib/Order/Filter/AtTopBot/Archimedean.lean,Mathlib/Order/Filter/AtTopBot/Field.lean |
2 |
1 |
['github-actions'] |
nobody |
2-30191 2 days ago |
2-30198 2 days ago |
2-32318 2 days |
29476 |
llllvvuu author:llllvvuu |
feat(LinearAlgebra/Matrix): `charpoly` splits into `IsHermitian.eigenvalues` |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
52/12 |
Mathlib/LinearAlgebra/Matrix/HermitianFunctionalCalculus.lean,Mathlib/LinearAlgebra/Matrix/Spectrum.lean |
2 |
7 |
['github-actions', 'llllvvuu', 'mathlib4-merge-conflict-bot', 'themathqueen'] |
j-loreaux assignee:j-loreaux |
2-25004 2 days ago |
2-33181 2 days ago |
3-54583 3 days |
29248 |
mans0954 author:mans0954 |
feature(Analysis/Convex/Basic): Convexity and the algebra map |
Let `R` and `A` be ordered rings, `A` an `R`-algebra and `R`, `A`, `M` a scalar tower. We provide sufficient conditions for an `R`-convex subset of `M` to be `A`-convex and for an `A`-convex subset of `M` to be `R`-convex.
These are used to show that, when `K` is `RCLike` and `ℝ` `K` `E` is a scalar tower, a set is `K`-convex if and only if it is `ℝ`-convex.
Used in #29258
---
[](https://gitpod.io/from-referrer/)
|
t-analysis |
49/0 |
Mathlib/Analysis/Convex/Basic.lean,Mathlib/Analysis/RCLike/Lemmas.lean |
2 |
4 |
['github-actions', 'mans0954'] |
j-loreaux assignee:j-loreaux |
2-21604 2 days ago |
10-63258 10 days ago |
10-63248 10 days |
29538 |
YaelDillies author:YaelDillies |
refactor(FractionalIdeal): use algebraic order theory API |
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
WIP
|
76/45 |
Mathlib/RingTheory/DedekindDomain/Different.lean,Mathlib/RingTheory/DedekindDomain/Ideal/Basic.lean,Mathlib/RingTheory/DedekindDomain/Ideal/Lemmas.lean,Mathlib/RingTheory/FractionalIdeal/Basic.lean,Mathlib/RingTheory/FractionalIdeal/Inverse.lean,Mathlib/RingTheory/FractionalIdeal/Operations.lean |
6 |
1 |
['github-actions'] |
nobody |
2-18237 2 days ago |
2-18238 2 days ago |
0-8 8 seconds |
29503 |
zhuyizheng author:zhuyizheng |
feat(MeasureTheory): add Lebesgue differentiation theorem for intervals |
Add the Lebesgue differentiation theorem for intervals. Part of originally planned #29092.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-measure-probability
|
77/0 |
Mathlib.lean,Mathlib/Analysis/Calculus/Deriv/Slope.lean,Mathlib/MeasureTheory/Integral/IntervalIntegral/LebesgueDifferetiationThm.lean |
3 |
19 |
['github-actions', 'themathqueen', 'vlad902'] |
nobody |
2-17843 2 days ago |
2-65865 2 days ago |
2-73149 2 days |
29426 |
kim-em author:kim-em |
feat: grind annotations for Finset.range |
------------------
- [x] depends on: #29509 |
t-data |
21/29 |
Mathlib/Data/Finset/Empty.lean,Mathlib/Data/Finset/Range.lean |
2 |
5 |
['eric-wieser', 'github-actions', 'kim-em', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
2-16640 2 days ago |
2-34823 2 days ago |
4-56709 4 days |
29539 |
YaelDillies author:YaelDillies |
feat: monoid algebras are invariant under base change |
From Toric
Co-authored-by: Michał Mrugała
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
toric
large-import
|
112/6 |
Mathlib.lean,Mathlib/Algebra/MonoidAlgebra/Basic.lean,Mathlib/RingTheory/TensorProduct/MonoidAlgebra.lean |
3 |
1 |
['github-actions'] |
nobody |
2-15963 2 days ago |
2-15963 2 days ago |
2-17370 2 days |
29510 |
sgouezel author:sgouezel |
chore: add missing fast_instance attributes |
---
[](https://gitpod.io/from-referrer/)
|
t-topology |
11/10 |
Mathlib/Topology/ContinuousMap/Bounded/Normed.lean,Mathlib/Topology/ContinuousMap/ZeroAtInfty.lean |
2 |
5 |
['github-actions', 'grunweg', 'leanprover-bot', 'themathqueen'] |
nobody |
2-15926 2 days ago |
2-66725 2 days ago |
2-66763 2 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
awaiting-author
|
24/0 |
Mathlib/Data/ENat/Lattice.lean |
1 |
5 |
['github-actions', 'kckennylau', 'mbkybky'] |
ericrbg assignee:ericrbg |
2-12649 2 days ago |
2-28533 2 days ago |
80-1250 80 days |
29324 |
tb65536 author:tb65536 |
refactor(Analysis/Calculus/IteratedDeriv/Defs): tweak statement of `iteratedDerivWithin_one` |
This PR removes the `x` from `iteratedDerivWithin_one` to make it match `iteratedDerivWithin_zero`.
---
[](https://gitpod.io/from-referrer/)
|
t-analysis |
3/2 |
Mathlib/Analysis/Calculus/IteratedDeriv/Defs.lean |
1 |
2 |
['github-actions', 'grunweg'] |
grunweg assignee:grunweg |
2-9890 2 days ago |
9-55035 9 days ago |
9-55017 9 days |
29247 |
harahu author:harahu |
doc: hyphenize "weighted homogeneous" when used attributively |
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
awaiting-author
|
18/18 |
Mathlib/RingTheory/MvPolynomial/EulerIdentity.lean,Mathlib/RingTheory/MvPolynomial/WeightedHomogeneous.lean,Mathlib/RingTheory/MvPowerSeries/Order.lean |
3 |
2 |
['chrisflav', 'github-actions'] |
chrisflav assignee:chrisflav |
2-8769 2 days ago |
2-8769 2 days ago |
8-67796 8 days |
29326 |
FormulaRabbit81 author:FormulaRabbit81 |
feat(Analysis): constant * function tending to 0 is still 0 |
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-analysis
|
24/0 |
Mathlib/Analysis/SpecificLimits/Basic.lean,Mathlib/Topology/Instances/ENNReal/Lemmas.lean,Mathlib/Topology/Instances/Real/Lemmas.lean |
3 |
2 |
['FormulaRabbit81', 'github-actions'] |
nobody |
2-6402 2 days ago |
2-6402 2 days ago |
9-59560 9 days |
29297 |
harahu author:harahu |
doc: hyphenate "first order" and "higher order" when used attributively |
Compound adjectives that are attributive (coming before their noun) should almost always be hyphenated in English.
This PR covers "first order" and "higher order".
---
[](https://gitpod.io/from-referrer/)
|
maintainer-merge |
24/24 |
Mathlib/Analysis/Calculus/ContDiff/FTaylorSeries.lean,Mathlib/Analysis/Fourier/FourierTransformDeriv.lean,Mathlib/FieldTheory/AxGrothendieck.lean,Mathlib/Logic/Basic.lean,Mathlib/ModelTheory/Algebra/Field/Basic.lean,Mathlib/ModelTheory/Algebra/Field/CharP.lean,Mathlib/ModelTheory/Algebra/Field/IsAlgClosed.lean,Mathlib/ModelTheory/Algebra/Ring/Basic.lean,Mathlib/RingTheory/MvPolynomial/FreeCommRing.lean,Mathlib/Topology/VectorBundle/Riemannian.lean,docs/undergrad.yaml |
11 |
3 |
['github-actions', 'grunweg'] |
nobody |
2-6314 2 days ago |
2-6314 2 days ago |
10-7959 10 days |
29256 |
harahu author:harahu |
doc: attach "quasi" as a prefix where it is currently freestanding |
---
[](https://gitpod.io/from-referrer/)
|
t-dynamics
t-measure-probability
|
25/25 |
Mathlib/AlgebraicGeometry/Morphisms/Descent.lean,Mathlib/Dynamics/BirkhoffSum/QuasiMeasurePreserving.lean,Mathlib/Dynamics/Ergodic/Ergodic.lean,Mathlib/Dynamics/Ergodic/Function.lean,Mathlib/GroupTheory/GroupAction/DomAct/Basic.lean,Mathlib/MeasureTheory/Function/AEEqFun.lean,Mathlib/MeasureTheory/Function/AEEqFun/DomAct.lean,Mathlib/MeasureTheory/Group/AEStabilizer.lean,Mathlib/MeasureTheory/Measure/QuasiMeasurePreserving.lean,Mathlib/MeasureTheory/Measure/Restrict.lean |
10 |
2 |
['MichaelStollBayreuth', 'github-actions'] |
nobody |
2-5052 2 days ago |
2-5124 2 days ago |
10-57809 10 days |
29430 |
RemyDegenne author:RemyDegenne |
refactor(Probability): change stopping times to take values in `WithTop` |
This PR changes stopping times to have type `Ω → WithTop ι` instead of `Ω → ι`.
Previously, a stopping time for a filtration indexed by Nat had to have value in Nat. That's not representative of the way stopping times are used in probability. A typical stopping time is the first time at which we see a head in an infinite sequence of coin flips. That time could be infinite (although it is almost surely finite). We can't represent it with a `Ω → Nat` stopping time: if we choose an arbitrary value in Nat for the event that it is infinite, we destroy the stopping time property.
We faced that issue in the `BorelCantelli` file, in which we avoided such a possibly infinite stopping time by introducing a sequence of bounded stopping times. We had to prove additional lemmas about them since we could not directly use the API for stopped processes. With the new type, that file is greatly simplified as the API is directly usable, and we can write the proof as we would on paper.
The issue with the previous stopping time implementation was noted in [Ying and Degenne, A Formalization of Doob’s Martingale Convergence Theorems in mathlib, CPP 2023, https://dl.acm.org/doi/pdf/10.1145/3573105.3575675].
Other changes:
- the sigma-algebra generated by a stopping time is now a sub-sigma algebra by definition
- `measurableSet_eq_stopping_time` is generalized and the now useless `measurableSet_eq_stopping_time_of_countable` is removed
- `hitting` is renamed to `hittingBtwn`
- a new `hittingAfter` is introduced and used in the Borel-Cantelli proof. That proof is now much simpler since we can use a stopped process as intended instead of going around the limitations of the previous stopping time implementation.
---
- [ ] depends on: #29466
[](https://gitpod.io/from-referrer/)
|
t-measure-probability
WIP
|
1090/556 |
Mathlib/Probability/Martingale/Basic.lean,Mathlib/Probability/Martingale/BorelCantelli.lean,Mathlib/Probability/Martingale/OptionalSampling.lean,Mathlib/Probability/Martingale/OptionalStopping.lean,Mathlib/Probability/Martingale/Upcrossing.lean,Mathlib/Probability/Process/HittingTime.lean,Mathlib/Probability/Process/Stopping.lean,Mathlib/Topology/Order/WithTop.lean |
8 |
10 |
['RemyDegenne', 'github-actions', 'kex-y', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
2-3709 2 days ago |
2-6100 2 days ago |
0-1 1 second |
29413 |
jsm28 author:jsm28 |
refactor(Geometry/Euclidean/Altitude,Geometry/Euclidean/Incenter): use `Nat.AtLeastTwo` |
Using `[Nat.AtLeastTwo n]` in place of `(hn : 1 < n)` saves passing various explicit hypotheses around, and is convenient in particular if applying lemmas in the common use case of a triangle.
As discussed on Zulip, `AtLeastTwo` is mainly used with literals at present, and there is no clear consensus about broader use in groups of lemmas sharing a common value of `n`, but `NeZero` is used in a similar way in the `rootsOfUnity` API.
---
[](https://gitpod.io/from-referrer/)
|
t-euclidean-geometry |
23/21 |
Mathlib/Geometry/Euclidean/Altitude.lean,Mathlib/Geometry/Euclidean/Incenter.lean |
2 |
4 |
['eric-wieser', 'github-actions', 'jsm28'] |
nobody |
2-1419 2 days ago |
5-46553 5 days ago |
5-46535 5 days |
29477 |
izanbf1803 author:izanbf1803 |
feat(Algebra/Ring/Invertible): add `eq_of_invOf_add_eq_invOf_add_invOf` |
Formalize statement and prove eq_of_invOf_add_eq_invOf_add_invOf
⅟(a + b) = ⅟a + ⅟b → a * ⅟b * a = b * ⅟a * b (for a, b in a ring; a, b invertible)
This will be useful to formalize a proof in https://github.com/eric-wieser/lean-matrix-cookbook.
|
new-contributor
t-algebra
label:t-algebra$ |
29/0 |
Mathlib/Algebra/Ring/Invertible.lean |
1 |
3 |
['eric-wieser', 'github-actions'] |
nobody |
2-730 2 days ago |
3-58583 3 days ago |
3-58628 3 days |
29552 |
RemyDegenne author:RemyDegenne |
feat(Probability): lemmas about composition of kernels and measures |
From the LeanBandits project.
---
[](https://gitpod.io/from-referrer/)
|
t-measure-probability |
44/0 |
Mathlib/Probability/ConditionalProbability.lean,Mathlib/Probability/Kernel/Composition/Lemmas.lean,Mathlib/Probability/Kernel/Composition/MeasureComp.lean,Mathlib/Probability/Kernel/Composition/ParallelComp.lean,Mathlib/Probability/Kernel/Composition/Prod.lean |
5 |
1 |
['github-actions'] |
nobody |
1-85614 1 day ago |
1-85624 1 day ago |
1-85662 1 day |
27098 |
Paul-Lez author:Paul-Lez |
feat(Algebra/Category/ModuleCat/Sheaf/VectorBundle): define vector bundles |
This PR defines vector bundles (upstreamed from [formal-conjectures](https://github.com/google-deepmind/formal-conjectures/pull/28/files)). I plan on adding some more API about the definition in this PR, but figured it would be nice to get some initial feedback about the definition before doing so!
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
awaiting-author
label:t-algebra$ |
53/0 |
Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Sheaf/VectorBundle.lean |
2 |
4 |
['Kiolt', 'Raph-DG', 'chrisflav', 'github-actions'] |
chrisflav assignee:chrisflav |
1-85213 1 day ago |
44-52894 1 month ago |
16-82639 16 days |
29554 |
RemyDegenne author:RemyDegenne |
feat(Probability): `CondIndepFun` lemmas |
Lemmas about conditional independence of constant random variables and of random variables that are measurable with respect to the sigma-algebra that we are conditioning on.
From the LeanBandits project.
---
[](https://gitpod.io/from-referrer/)
|
t-measure-probability |
94/2 |
Mathlib/Probability/Independence/Basic.lean,Mathlib/Probability/Independence/Conditional.lean,Mathlib/Probability/Independence/Kernel.lean |
3 |
1 |
['github-actions'] |
nobody |
1-84643 1 day ago |
1-84652 1 day ago |
1-84689 1 day |
29556 |
joelriou author:joelriou |
feat(CategoryTheory): canonical colimits |
Given a functor `F : C ⥤ D` and `Y : D`, we say that `Y` is a canonical colimit relatively to `F` is `Y` identifies to the colimit of all `F.obj X` for `X : C` and `f : F.obj X ⟶ Y`, i.e. `Y` identifies to the colimit of the obvious functor `CostructuredArrow F Y ⥤ D` (see definitions `canonicalCocone` and `CanonicalColimit`). We introduce the corresponding property `isCanonicalColimit F` of objects of `D`.
---
[](https://gitpod.io/from-referrer/)
|
t-category-theory |
72/0 |
Mathlib.lean,Mathlib/CategoryTheory/Limits/Canonical.lean |
2 |
1 |
['github-actions'] |
nobody |
1-82017 1 day ago |
1-82087 1 day ago |
1-82068 1 day |
25735 |
robin-carlier author:robin-carlier |
feat(CategoryTheory/Limits/Sifted): characterization of sifted categories |
Characterize small sifted as those for which the `Type`-valued colimit functor preserves finite product. Deduce that filtered categories, and that categories admitting a final functor from a sifted categories are also sifted.
---
Second part of what used to be #17554. The core of the proof relies on a few private lemmas/defs (`colimBoxIsoColimTensColim` and `factorization_prod_comparison_colim` being the most important ones) and I don’t know if that can be avoided.
I am still unsure wether or not the part relating sifted categories to filtered categories should be split off in a different file to avoid importing `CategoryTheory/Limits/FilteredColimitCommutesFiniteLimit.lean` every time `CategoryTheory/Limits/Sifted.lean` is imported.
The fact that filtered categories are sifted can also be proved without the characterization in this PR (it reduces essentially to `IsFiltered.bowtie`), and so it could also stay in this file with less imports, but I find it nicer to do it using the characterization.
- [x] depends on: #17766
- [x] depends on: #17779
- [x] depends on: #25732
- [x] depends on: #25734
- [x] depends on: #25731
- [x] depends on: #24735
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #17781.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/17781* |
large-import
t-category-theory
|
166/3 |
Mathlib/CategoryTheory/Limits/Indization/FilteredColimits.lean,Mathlib/CategoryTheory/Limits/Sifted.lean |
2 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
adamtopaz assignee:adamtopaz |
1-81883 1 day ago |
27-2275 27 days ago |
27-2283 27 days |
29482 |
mattrobball author:mattrobball |
refactor (Algebra.Group.Defs): add npow/zpow/nsmul/zsmul as fields of new parents classes |
Adds ZPow G class and makes this a parent to DivInvMonoid and the corresponding additive versions. Updates zpow/zsmul operations to use the integrated power/scalar multiplication syntax.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
177/122 |
Mathlib/Algebra/Group/Action/Defs.lean,Mathlib/Algebra/Group/Basic.lean,Mathlib/Algebra/Group/Commute/Defs.lean,Mathlib/Algebra/Group/Defs.lean,Mathlib/Algebra/Group/Ext.lean,Mathlib/Algebra/Group/Int/Defs.lean,Mathlib/Algebra/Group/Opposite.lean,Mathlib/Algebra/Group/Pointwise/Set/Basic.lean,Mathlib/Algebra/Group/Prod.lean,Mathlib/Algebra/Group/Submonoid/Membership.lean,Mathlib/Algebra/Group/TypeTags/Basic.lean,Mathlib/Algebra/Group/Units/Defs.lean,Mathlib/Algebra/GroupWithZero/Basic.lean,Mathlib/Algebra/Module/NatInt.lean,Mathlib/Algebra/Order/GroupWithZero/Unbundled/Basic.lean,Mathlib/Algebra/Order/Monoid/Unbundled/WithTop.lean,Mathlib/Algebra/Order/Ring/Unbundled/Basic.lean,Mathlib/Algebra/Ring/ULift.lean,Mathlib/Data/BitVec.lean,Mathlib/Tactic/Abel.lean,Mathlib/Tactic/NormNum/Pow.lean |
21 |
1 |
['github-actions'] |
nobody |
1-78058 1 day ago |
3-47989 3 days ago |
0-0 0 seconds |
29550 |
Raph-DG author:Raph-DG |
feat(RingTheory): Order of vanishing in a discrete valuation ring |
In this PR we develop some API for working with the order of vanishing in a discrete valuation ring.
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
file-removed
|
462/1 |
Mathlib.lean,Mathlib/RingTheory/DiscreteValuationRing/Basic.lean,Mathlib/RingTheory/OrderOfVanishing/Basic.lean,Mathlib/RingTheory/OrderOfVanishing/Properties.lean |
4 |
1 |
['github-actions'] |
nobody |
1-75151 1 day ago |
1-86198 1 day ago |
1-86250 1 day |
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 |
63 |
['FLDutchmann', 'Paul-Lez', 'YaelDillies', 'eric-wieser', 'github-actions', 'grunweg', 'kckennylau', 'kim-em', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'urkud'] |
eric-wieser assignee:eric-wieser |
1-74656 1 day ago |
150-1621 4 months ago |
205-48737 205 days |
28266 |
euprunin author:euprunin |
chore(RingTheory): golf entire `single_one_eq_pow` using `simp` |
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
awaiting-author
|
1/5 |
Mathlib/RingTheory/LaurentSeries.lean |
1 |
6 |
['eric-wieser', 'github-actions', 'grunweg', 'mathlib4-merge-conflict-bot'] |
nobody |
1-70149 1 day ago |
1-70167 1 day ago |
0-11379 3 hours |
29547 |
kim-em author:kim-em |
chore: remove defunct polyrith tactic |
In my understanding, the public Sage server that `polyrith` relies on is down and never going to come back, and hence the `polyrith` code is dead. There are a bunch of viable options for restoring this, e.g. running Sage locally, running our own Sage server, moving to a different external CAS, implementing Grobner bases in a way that produces nullstellensatz certificates (including by modifying the `grind` implementation). But none of these exist at the moment, so this code in Mathlib is not of any use. It can immediately be restored from history if someone wants to implement one of these solutions. In the meantime, one can also use `grobner` (which calls the Grobner module in `grind`) to close the goal without a source code certificate. |
file-removed |
16/1235 |
Archive/Imo/Imo1962Q4.lean,Archive/Imo/Imo2006Q3.lean,Mathlib/Algebra/Star/CHSH.lean,Mathlib/Tactic/Polyrith.lean,MathlibTest/polyrith.lean,scripts/README.md,scripts/noshake.json,scripts/polyrith_sage_helper.py |
8 |
2 |
['euprunin', 'github-actions', 'kim-em'] |
nobody |
1-69923 1 day ago |
2-2842 2 days ago |
2-2891 2 days |
29536 |
kim-em author:kim-em |
chore: minor grind golfing in Logic/Embedding |
---
[](https://gitpod.io/from-referrer/)
|
maintainer-merge
t-logic
|
18/14 |
Mathlib/Logic/Embedding/Basic.lean,Mathlib/Logic/Embedding/Set.lean |
2 |
2 |
['euprunin', 'github-actions', 'grunweg'] |
nobody |
1-69886 1 day ago |
2-5671 2 days ago |
2-25374 2 days |
29492 |
kim-em author:kim-em |
feat: grind golf in Mathlib.Data.List |
Much of this comes from locations identified by the new `linter.tacticAnalysis.terminalToGrind`, and then cleaning up in flagged files. |
t-data |
74/231 |
Mathlib/Data/List/Basic.lean,Mathlib/Data/List/Flatten.lean,Mathlib/Data/List/Induction.lean,Mathlib/Data/List/Lattice.lean,Mathlib/Data/List/Lookmap.lean,Mathlib/Data/List/ReduceOption.lean,Mathlib/Data/List/SplitOn.lean,Mathlib/Data/List/TakeDrop.lean,Mathlib/Data/List/Triplewise.lean,Mathlib/Data/Multiset/UnionInter.lean |
10 |
5 |
['eric-wieser', 'euprunin', 'github-actions', 'kim-em'] |
nobody |
1-69724 1 day ago |
3-15349 3 days ago |
3-15394 3 days |
26479 |
thefundamentaltheor3m author:thefundamentaltheor3m |
feat(Analysis/Complex/CauchyIntegral): Cauchy-Goursat for Unbounded Rectangles |
In this PR, we prove versions of the Cauchy-Goursat theorem where the contours in question are rectangular and unbounded (ie, where the contours look like the $\bigsqcup$ symbol). I am not sure if I have formalised these in the best way, or if `Analysis.Complex.CauchyIntegral` is the best place for them (it might be prudent to reorganise the file into multiple files at some point), but I believe this is a useful result. Suggestions welcome.
---
[](https://gitpod.io/from-referrer/)
|
large-import
new-contributor
t-analysis
|
201/0 |
Mathlib/Analysis/Complex/CauchyIntegral.lean |
1 |
1 |
['github-actions'] |
nobody |
1-69687 1 day ago |
77-67636 2 months ago |
0-0 0 seconds |
25778 |
thefundamentaltheor3m author:thefundamentaltheor3m |
feat: Monotonicity of `setIntegral` for nonnegative functions |
This PR makes it easier to prove monotonicity of the Bochner integral on sets for nonnegative functions by removing the stronger assumption required by the general monotonicity lemma that both of the functions being compared must be integrable.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-measure-probability
awaiting-author
|
8/0 |
Mathlib/MeasureTheory/Integral/Bochner/Set.lean |
1 |
6 |
['RemyDegenne', 'github-actions', 'sgouezel', 'thefundamentaltheor3m'] |
nobody |
1-69687 1 day ago |
92-77520 3 months ago |
0-11893 3 hours |
29562 |
ShreckYe author:ShreckYe |
feat(Analysis/SpecialFunctions/Trigonometric): tangent half-angle substitution |
|
t-analysis |
82/0 |
Mathlib/Analysis/SpecialFunctions/Trigonometric/Complex.lean |
1 |
1 |
['github-actions'] |
nobody |
1-66147 1 day ago |
1-66159 1 day ago |
1-66203 1 day |
27847 |
euprunin author:euprunin |
chore(Algebra): avoid duplicating proofs by reusing existing theorems or lemmas |
|
t-algebra label:t-algebra$ |
46/73 |
Archive/Imo/Imo1972Q5.lean,Archive/Imo/Imo2015Q6.lean,Mathlib/Algebra/Homology/Embedding/Extend.lean,Mathlib/Algebra/MvPolynomial/Rename.lean,Mathlib/Algebra/Order/AbsoluteValue/Basic.lean,Mathlib/Algebra/Order/Archimedean/Class.lean,Mathlib/Algebra/Order/BigOperators/Expect.lean,Mathlib/Algebra/Order/BigOperators/Group/Finset.lean,Mathlib/Algebra/Order/BigOperators/Group/Multiset.lean,Mathlib/Algebra/Order/Group/Abs.lean,Mathlib/Algebra/Order/Ring/Unbundled/Rat.lean,Mathlib/Algebra/Polynomial/Degree/Lemmas.lean,Mathlib/Algebra/Polynomial/Monic.lean,Mathlib/AlgebraicGeometry/EllipticCurve/DivisionPolynomial/Degree.lean,Mathlib/Analysis/MeanInequalities.lean,Mathlib/Analysis/Normed/Lp/lpSpace.lean,Mathlib/Data/NNRat/Defs.lean,Mathlib/MeasureTheory/Function/Jacobian.lean,Mathlib/NumberTheory/Pell.lean,Mathlib/RingTheory/Polynomial/Basic.lean,Mathlib/Tactic/ComputeDegree.lean,Mathlib/Topology/Algebra/Order/Group.lean,Mathlib/Topology/MetricSpace/Algebra.lean,MathlibTest/GCongr/inequalities.lean,MathlibTest/GRewrite.lean |
25 |
18 |
['Ruben-VandeVelde', 'euprunin', 'github-actions', 'grunweg', 'kbuzzard', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'mathlib4-merge-conflict-bot'] |
mariainesdff assignee:mariainesdff |
1-64873 1 day ago |
1-64873 1 day ago |
39-4783 39 days |
25930 |
loefflerd author:loefflerd |
WIP towards Hecke bound for q-expansions |
The aim of this PR is to prove various statements about boundedness properties of modular forms.
---
This PR continues the work from #24962.
Original PR: https://github.com/leanprover-community/mathlib4/pull/24962 |
migrated-from-branch
t-number-theory
WIP
|
789/138 |
Mathlib.lean,Mathlib/NumberTheory/ModularForms/Bounds.lean,Mathlib/NumberTheory/ModularForms/CongruenceSubgroups.lean,Mathlib/NumberTheory/ModularForms/EisensteinSeries/IsBoundedAtImInfty.lean,Mathlib/NumberTheory/ModularForms/Identities.lean,Mathlib/NumberTheory/ModularForms/LevelOne.lean,Mathlib/NumberTheory/ModularForms/Petersson.lean,Mathlib/NumberTheory/ModularForms/QExpansion.lean |
8 |
4 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-merge-conflict-bot'] |
nobody |
1-62591 1 day ago |
17-5274 17 days ago |
0-77 1 minute |
29563 |
j-loreaux author:j-loreaux |
refactor: switch to using `Fact (0 ∈ s)` for `ContinuousMapZero.id` |
`ContinuousMapZero` is used exclusively for the non-unital continuous functional calculus. Within this scope we have an instance `Zero s` for `s : Set R` under the assumption `Fact (0 ∈ s)`. This is somewhat reasonable because, in the most common scenario, `s := quasispectrum R a`, for which we can always provide this `Fact` instance.
However, several declarations were put in place prior to this `Zero` instance, and they made use of a different paradigm where we take `Zero s` as an *argument* and then have another argument of the form `h0 : ↑(0 : s) = (0 : R)`. This PR shifts that paradigm into the new regime, and I think this change is beneficial.
---
[](https://gitpod.io/from-referrer/)
|
t-analysis |
69/79 |
Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Basic.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Continuity.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Instances.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/NonUnital.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Restrict.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Unique.lean,Mathlib/Analysis/SpecialFunctions/ContinuousFunctionalCalculus/PosPart/Basic.lean,Mathlib/Topology/ContinuousMap/ContinuousMapZero.lean,Mathlib/Topology/ContinuousMap/StoneWeierstrass.lean |
9 |
2 |
['github-actions', 'j-loreaux'] |
nobody |
1-62216 1 day ago |
1-62387 1 day ago |
1-62377 1 day |
28035 |
euprunin author:euprunin |
chore: replace `norm_num` with `simp` where applicable |
Same motivation as in kim-em's #24064 (chore: replace `norm_num` with `simp` where applicable):
> Consider replacing a tactic with a (ahem) simpler alternative.
Note that `norm_num` runs `simp` internally, so using `simp` is simply faster.
|
|
156/157 |
Mathlib/Algebra/Polynomial/Div.lean,Mathlib/Algebra/Star/CHSH.lean,Mathlib/AlgebraicTopology/FundamentalGroupoid/Basic.lean,Mathlib/Analysis/Analytic/Inverse.lean,Mathlib/Analysis/Asymptotics/AsymptoticEquivalent.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Order.lean,Mathlib/Analysis/Calculus/Deriv/MeanValue.lean,Mathlib/Analysis/Calculus/Taylor.lean,Mathlib/Analysis/Complex/Trigonometric.lean,Mathlib/Analysis/ConstantSpeed.lean,Mathlib/Analysis/Convex/Function.lean,Mathlib/Analysis/Fourier/AddCircle.lean,Mathlib/Analysis/Fourier/Inversion.lean,Mathlib/Analysis/Fourier/RiemannLebesgueLemma.lean,Mathlib/Analysis/InnerProductSpace/Basic.lean,Mathlib/Analysis/InnerProductSpace/LinearMap.lean,Mathlib/Analysis/InnerProductSpace/Orthonormal.lean,Mathlib/Analysis/InnerProductSpace/TwoDim.lean,Mathlib/Analysis/NormedSpace/ENormedSpace.lean,Mathlib/Analysis/PSeries.lean,Mathlib/Analysis/Real/Cardinality.lean,Mathlib/Analysis/Real/Pi/Bounds.lean,Mathlib/Analysis/SpecialFunctions/Complex/LogBounds.lean,Mathlib/Analysis/SpecialFunctions/ContinuousFunctionalCalculus/Rpow/Basic.lean,Mathlib/Analysis/SpecialFunctions/Gamma/Beta.lean,Mathlib/Analysis/SpecialFunctions/Gamma/BohrMollerup.lean,Mathlib/Analysis/SpecialFunctions/Gaussian/GaussianIntegral.lean,Mathlib/Analysis/SpecialFunctions/Integrals/Basic.lean,Mathlib/Analysis/SpecialFunctions/Integrals/PosLogEqCircleAverage.lean,Mathlib/Analysis/SpecialFunctions/JapaneseBracket.lean,Mathlib/Analysis/SpecialFunctions/Pow/Real.lean,Mathlib/Analysis/SpecialFunctions/Stirling.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Basic.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Bounds.lean,Mathlib/Analysis/SpecificLimits/Normed.lean,Mathlib/Combinatorics/Additive/AP/Three/Behrend.lean,Mathlib/Combinatorics/Additive/SmallTripling.lean,Mathlib/Combinatorics/SimpleGraph/Regularity/Bound.lean,Mathlib/Combinatorics/SimpleGraph/Regularity/Chunk.lean,Mathlib/Combinatorics/SimpleGraph/Regularity/Lemma.lean,Mathlib/Computability/Ackermann.lean,Mathlib/Computability/AkraBazzi/SumTransform.lean,Mathlib/Data/EReal/Basic.lean,Mathlib/Data/Nat/Digits/Div.lean,Mathlib/Data/Real/GoldenRatio.lean,Mathlib/Data/Real/Sign.lean,Mathlib/Geometry/Euclidean/Basic.lean,Mathlib/Geometry/Euclidean/MongePoint.lean,Mathlib/Geometry/Euclidean/Triangle.lean,Mathlib/GroupTheory/GroupAction/Blocks.lean,Mathlib/GroupTheory/Perm/Cycle/Basic.lean,Mathlib/GroupTheory/SpecificGroups/Alternating/KleinFour.lean,Mathlib/GroupTheory/SpecificGroups/Quaternion.lean,Mathlib/LinearAlgebra/QuadraticForm/Basic.lean,Mathlib/LinearAlgebra/RootSystem/Reduced.lean,Mathlib/MeasureTheory/Function/ConvergenceInMeasure.lean,Mathlib/MeasureTheory/Function/UniformIntegrable.lean,Mathlib/MeasureTheory/Integral/Bochner/Basic.lean,Mathlib/MeasureTheory/Integral/CircleIntegral.lean,Mathlib/NumberTheory/ADEInequality.lean,Mathlib/NumberTheory/Bernoulli.lean,Mathlib/NumberTheory/Cyclotomic/Discriminant.lean,Mathlib/NumberTheory/Cyclotomic/PID.lean,Mathlib/NumberTheory/Cyclotomic/Rat.lean,Mathlib/NumberTheory/FactorisationProperties.lean,Mathlib/NumberTheory/Fermat.lean,Mathlib/NumberTheory/FermatPsp.lean,Mathlib/NumberTheory/Harmonic/GammaDeriv.lean,Mathlib/NumberTheory/Harmonic/ZetaAsymp.lean,Mathlib/NumberTheory/LSeries/DirichletContinuation.lean,Mathlib/NumberTheory/LucasLehmer.lean,Mathlib/NumberTheory/Modular.lean,Mathlib/NumberTheory/ModularForms/Basic.lean,Mathlib/NumberTheory/ModularForms/LevelOne.lean,Mathlib/NumberTheory/Multiplicity.lean,Mathlib/NumberTheory/NumberField/CanonicalEmbedding/ConvexBody.lean,Mathlib/NumberTheory/NumberField/Discriminant/Basic.lean,Mathlib/NumberTheory/NumberField/Discriminant/Defs.lean,Mathlib/NumberTheory/Padics/Hensel.lean,Mathlib/NumberTheory/Zsqrtd/GaussianInt.lean,Mathlib/RingTheory/DedekindDomain/Different.lean,Mathlib/RingTheory/Fintype.lean,Mathlib/RingTheory/Ideal/NatInt.lean,Mathlib/RingTheory/PowerSeries/Basic.lean,Mathlib/RingTheory/ZMod/UnitsCyclic.lean,Mathlib/Tactic/NormNum/LegendreSymbol.lean,Mathlib/Topology/Algebra/Valued/WithZeroMulInt.lean,Mathlib/Topology/Instances/CantorSet.lean,Mathlib/Topology/Instances/ENNReal/Lemmas.lean,Mathlib/Topology/Separation/CompletelyRegular.lean |
90 |
22 |
['github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
1-62174 1 day ago |
1-66384 1 day ago |
36-84078 36 days |
26640 |
euprunin author:euprunin |
chore(Data): golf `Data/` using `grind` |
|
bench-after-CI
t-data
|
10/78 |
Mathlib/Data/EReal/Operations.lean,Mathlib/Data/List/Cycle.lean,Mathlib/Data/List/Induction.lean,Mathlib/Data/List/Nodup.lean,Mathlib/Data/List/Sigma.lean,Mathlib/Data/PEquiv.lean,Mathlib/Data/PNat/Xgcd.lean,Mathlib/Data/Prod/Lex.lean,Mathlib/Data/Set/Lattice.lean |
9 |
29 |
['euprunin', 'github-actions', 'grunweg', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
1-62142 1 day ago |
1-70094 1 day ago |
70-29404 70 days |
28996 |
euprunin author:euprunin |
chore: remove redundant `have`:s in `Computability/`, `Combinatorics/`, `Condensed/`, `Data/Nat/` and `Data/PNat/` |
---
[](https://gitpod.io/from-referrer/)
|
|
0/12 |
Mathlib/Computability/AkraBazzi/AkraBazzi.lean,Mathlib/Computability/DFA.lean,Mathlib/Condensed/AB.lean,Mathlib/Data/Nat/BitIndices.lean,Mathlib/Data/Nat/Init.lean,Mathlib/Data/PNat/Xgcd.lean |
6 |
11 |
['JovanGerb', 'euprunin', 'github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'mathlib4-merge-conflict-bot'] |
JovanGerb assignee:JovanGerb |
1-61851 1 day ago |
1-61851 1 day ago |
16-58425 16 days |
29564 |
dagurtomas author:dagurtomas |
feat(CategoryTheory/Monoidal): more natural constructors for monoidal functors |
---
[](https://gitpod.io/from-referrer/)
|
t-category-theory |
523/0 |
Mathlib.lean,Mathlib/CategoryTheory/Monoidal/Multifunctor.lean |
2 |
1 |
['github-actions'] |
nobody |
1-61703 1 day ago |
1-61721 1 day ago |
1-61768 1 day |
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
delegated
|
96/120 |
Archive/Wiedijk100Theorems/AscendingDescendingSequences.lean |
1 |
13 |
['b-mehta', 'github-actions', 'grunweg', 'j-loreaux', 'mathlib-bors'] |
ericrbg assignee:ericrbg |
1-61520 1 day ago |
1-61520 1 day ago |
78-81111 78 days |
29540 |
YaelDillies author:YaelDillies |
refactor(SimpleGraph): make `triangleRemovalBound` positive more often |
It wasn't positive when `ε > 4`, but that is a junk value anyway, so we change the junk value to a positive one.
See #29496 for more context.
---
[](https://gitpod.io/from-referrer/)
|
t-combinatorics |
66/40 |
Mathlib/Combinatorics/Additive/Corner/Roth.lean,Mathlib/Combinatorics/SimpleGraph/DeleteEdges.lean,Mathlib/Combinatorics/SimpleGraph/Triangle/Basic.lean,Mathlib/Combinatorics/SimpleGraph/Triangle/Removal.lean,Mathlib/Data/Nat/Choose/Bounds.lean,Mathlib/Data/Nat/Factorial/Basic.lean |
6 |
3 |
['github-actions', 'grunweg'] |
grunweg assignee:grunweg |
1-61004 1 day ago |
1-61065 1 day ago |
1-64222 1 day |
26955 |
mariainesdff author:mariainesdff |
feat(LinearAlgebra/OnSup): extend linear maps to sums of modules |
Let `A` be a ring, `X, Y` be `A`-modules, and `M, N` be `A`-submodules of `X`.
Given two linear maps `f : M →ₗ[A] Y` and `g : N →ₗ[A] Y` that agree on `M ∩ N`, there is a unique linear map `M + N →ₗ[A] Y` that simultaneously extends `f` and `g`.
Co-authored-by: @AntoineChambert-Loir
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
awaiting-author
label:t-algebra$ |
153/0 |
Mathlib.lean,Mathlib/LinearAlgebra/OnSup.lean |
2 |
16 |
['AntoineChambert-Loir', 'eric-wieser', 'github-actions', 'j-loreaux', 'wwylele'] |
alreadydone assignee:alreadydone |
1-60982 1 day ago |
1-60982 1 day ago |
59-73968 59 days |
27864 |
BoltonBailey author:BoltonBailey |
feat(Data/{Finset,Multiset}/Sort): give sort functions ≤ default argument |
Changes the `Finset.sort` and `Multiset.sort` functions to take `≤` as the default relation argument. Then removes this argument where possible through the rest of the library.
This involves switching the order of arguments, but I think this is fine, as this function is mostly called by dot notation anyway, and I think it is more typical for the first argument of such functions to have the type that matches the namespace.
Thanks to @eric-wieser for suggesting this approach
Zulip discussion: [#mathlib4 > Redefine {Fin/Multi}set.sort to take linear order?](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Redefine.20.7BFin.2FMulti.7Dset.2Esort.20to.20take.20linear.20order.3F/with/532398325)
---
[](https://gitpod.io/from-referrer/)
|
t-data |
121/97 |
Mathlib/Algebra/Polynomial/Basic.lean,Mathlib/Data/Finset/Sort.lean,Mathlib/Data/Multiset/Sort.lean,Mathlib/Data/Nat/Nth.lean,Mathlib/GroupTheory/Perm/Cycle/Factors.lean,Mathlib/GroupTheory/Perm/Sign.lean,Mathlib/Logic/Equiv/Finset.lean,Mathlib/Logic/Equiv/Multiset.lean,Mathlib/NumberTheory/ADEInequality.lean |
9 |
5 |
['BoltonBailey', 'eric-wieser', 'github-actions', 'grunweg'] |
nobody |
1-60593 1 day ago |
41-69637 1 month ago |
42-36774 42 days |
29530 |
ShreckYe author:ShreckYe |
feat(Dynamics/PeriodicPts): some theorems for `Pi.map` in `Dynamics/PeriodicPts` analogous to those for `Prod.map` |
Split from #29204. Some namespace prefixes are added in `GroupTheory/OrderOfElement.lean` to distinguish the extra imports introduced.
- [ ] depends on: #29528
|
large-import |
77/8 |
Mathlib/Dynamics/PeriodicPts/Defs.lean,Mathlib/Dynamics/PeriodicPts/Lemmas.lean,Mathlib/GroupTheory/OrderOfElement.lean |
3 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
1-60355 1 day ago |
1-60738 1 day ago |
1-61395 1 day |
29395 |
YaelDillies author:YaelDillies |
refactor: make `PosMulMono` and alike custom classes |
In the current setup, users get confusing non-beta-reduced goals involving a subtype when trying to provide an instance of `PosMulMono`.
This PR changes it to be a custom structure with the expected fields.
This follows `PosSMulMono` and alike.
---
[](https://gitpod.io/from-referrer/)
|
t-order
t-algebra
label:t-algebra$ |
181/260 |
Counterexamples/CanonicallyOrderedCommSemiringTwoMul.lean,Mathlib/Algebra/Algebra/Operations.lean,Mathlib/Algebra/Order/GroupWithZero/Canonical.lean,Mathlib/Algebra/Order/GroupWithZero/Unbundled/Basic.lean,Mathlib/Algebra/Order/GroupWithZero/Unbundled/Defs.lean,Mathlib/Algebra/Order/GroupWithZero/WithZero.lean,Mathlib/Algebra/Order/Pi.lean,Mathlib/Algebra/Order/Ring/Canonical.lean,Mathlib/Algebra/Order/Ring/Defs.lean,Mathlib/Algebra/Order/Ring/InjSurj.lean,Mathlib/Algebra/Order/Ring/Nat.lean,Mathlib/Algebra/Order/Ring/Opposite.lean,Mathlib/Algebra/Order/Ring/Prod.lean,Mathlib/Algebra/Order/Ring/Star.lean,Mathlib/Algebra/Order/Ring/WithTop.lean,Mathlib/Data/NNRat/Defs.lean,Mathlib/Data/Num/Lemmas.lean,Mathlib/Order/Filter/FilterProduct.lean,Mathlib/Order/Filter/Ring.lean,Mathlib/SetTheory/Ordinal/Arithmetic.lean,Mathlib/SetTheory/Ordinal/NaturalOps.lean,MathlibTest/GRewrite.lean |
22 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
1-58588 1 day ago |
1-58588 1 day ago |
1-58601 1 day |
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 |
156/99 |
Mathlib/Algebra/Order/GroupWithZero/Canonical.lean,Mathlib/Algebra/Order/Monoid/Unbundled/WithTop.lean,Mathlib/Analysis/Analytic/OfScalars.lean,Mathlib/Analysis/Oscillation.lean,Mathlib/Data/Finset/Lattice/Fold.lean,Mathlib/Data/Finset/Max.lean,Mathlib/LinearAlgebra/Eigenspace/Triangularizable.lean,Mathlib/MeasureTheory/Integral/Lebesgue/Countable.lean,Mathlib/MeasureTheory/Measure/LevyProkhorovMetric.lean,Mathlib/Order/Interval/Basic.lean,Mathlib/Order/Interval/Set/WithBotTop.lean,Mathlib/Order/KrullDimension.lean,Mathlib/Order/WithBot.lean,Mathlib/Probability/Moments/Variance.lean,Mathlib/RingTheory/PowerBasis.lean,Mathlib/Topology/MetricSpace/Holder.lean,Mathlib/Topology/MetricSpace/HolderNorm.lean,MathlibTest/hint.lean |
18 |
23 |
['JovanGerb', 'YaelDillies', 'b-mehta', 'eric-wieser', 'github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'urkud'] |
Vierkantor assignee:Vierkantor |
1-58103 1 day ago |
2-11227 2 days ago |
168-41174 168 days |
26398 |
ChrisHughes24 author:ChrisHughes24 |
feat(ModelTheory): definable functions |
---
Possibly this should be generalized to partial functions.
I migrated the PR by hand instead of using the script.
- [x] depends on: #20166
- [x] depends on: #20161
- [x] depends on: #20115
- [x] depends on: #20174
- [x] depends on: #20175
- [x] depends on: #21948
[](https://gitpod.io/from-referrer/)
|
t-logic |
618/0 |
Mathlib.lean,Mathlib/ModelTheory/FunctionalFormula.lean |
2 |
7 |
['ChrisHughes24', 'github-actions', 'kckennylau', 'mathlib4-dependent-issues-bot'] |
fpvandoorn assignee:fpvandoorn |
1-57994 1 day ago |
80-5782 2 months ago |
80-6037 80 days |
26720 |
vlad902 author:vlad902 |
feat(SimpleGraph): lemmas relating edges and darts to the support |
Useful lemmas to make it easier to pass between the support/edges/darts of a walk.
- [ ] depends on: #25812
---
[](https://gitpod.io/from-referrer/)
|
t-combinatorics |
27/0 |
Mathlib/Combinatorics/SimpleGraph/Walk.lean |
1 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
1-57423 1 day ago |
1-64330 1 day ago |
1-64413 1 day |
26785 |
TOMILO87 author:TOMILO87 |
feat: beta distribution |
Add the Beta distribution to the probability distributions in mathlib4
This PR introduces the Beta distribution on the reals.
Main definitions:
- betaPDFReal (α β x : ℝ) — the probability density function as a real-valued function
- betaPDF (α β x : ℝ) — the pdf as a ℝ≥0∞-valued function
- betaMeasure (α β : ℝ) — the probability measure associated with the Beta distribution
Main results:
- lintegral_betaPDF_eq_one — proof that the pdf integrates to 1 (normalization)
- Lemmas on positivity, measurability, and integrability of the pdf
- isProbabilityMeasureBeta — the Beta measure is a probability measure
Notes:
- Follows the general structure of other distributions in mathlib (e.g. Gamma).
- Several unused helper lemmas were removed, and proofs streamlined in response to reviewer feedback.
- Thanks to @EtienneC30 and @RemyDegenne for detailed reviews across multiple rounds.
This is a clean version of the PR originally opened as [#25608](https://github.com/leanprover-community/mathlib4/pull/25608) and temporarily migrated in [#26325](https://github.com/leanprover-community/mathlib4/pull/26325).
|
new-contributor
t-measure-probability
|
206/2 |
Mathlib.lean,Mathlib/Algebra/Polynomial/Basic.lean,Mathlib/Analysis/SpecialFunctions/Gamma/Beta.lean,Mathlib/Probability/Distributions/Beta.lean |
4 |
34 |
['EtienneC30', 'RemyDegenne', 'TOMILO87', 'github-actions'] |
EtienneC30 assignee:EtienneC30 |
1-57300 1 day ago |
28-281 28 days ago |
59-13032 59 days |
29463 |
HugLycan author:HugLycan |
feat(Positivity): add positivity extensions for `NNReal.rpow` and `ENNReal.rpow` |
---
This PR adds positivity extensions for `NNReal.rpow` and `ENNReal.rpow`.
related issue #6038
@fpvandoorn
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-analysis
awaiting-author
|
76/3 |
Mathlib/Analysis/SpecialFunctions/Pow/NNReal.lean,MathlibTest/positivity.lean |
2 |
3 |
['HugLycan', 'github-actions', 'grunweg'] |
nobody |
1-56855 1 day ago |
4-4075 4 days ago |
0-1704 28 minutes |
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 |
4 |
['b-mehta', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-merge-conflict-bot'] |
adomani assignee:adomani |
1-55484 1 day ago |
1-62279 1 day ago |
85-62326 85 days |
29295 |
YaelDillies author:YaelDillies |
chore: rename `mul_lt_mul_left`/`mul_lt_mul_right` to `mul_lt_mul_iff_right₀`/`mul_lt_mul_iff_left₀` |
Follow up to #28645
---
[](https://gitpod.io/from-referrer/)
|
t-order
t-algebra
label:t-algebra$ |
108/114 |
Archive/Imo/Imo2011Q3.lean,Counterexamples/CanonicallyOrderedCommSemiringTwoMul.lean,Mathlib/Algebra/Order/Archimedean/Basic.lean,Mathlib/Algebra/Order/GroupWithZero/Unbundled/Basic.lean,Mathlib/Algebra/Order/GroupWithZero/Unbundled/Defs.lean,Mathlib/Algebra/Order/GroupWithZero/WithZero.lean,Mathlib/Algebra/Polynomial/Eval/Degree.lean,Mathlib/Analysis/BoxIntegral/UnitPartition.lean,Mathlib/Analysis/Convex/Slope.lean,Mathlib/Analysis/Fourier/RiemannLebesgueLemma.lean,Mathlib/Analysis/Normed/Group/AddCircle.lean,Mathlib/Analysis/Normed/Unbundled/SpectralNorm.lean,Mathlib/Analysis/Real/Cardinality.lean,Mathlib/Analysis/Seminorm.lean,Mathlib/Analysis/SpecialFunctions/BinaryEntropy.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Arctan.lean,Mathlib/Combinatorics/SimpleGraph/Regularity/Lemma.lean,Mathlib/Combinatorics/SimpleGraph/Triangle/Basic.lean,Mathlib/Computability/Ackermann.lean,Mathlib/Data/NNReal/Defs.lean,Mathlib/Data/Nat/Choose/Central.lean,Mathlib/Data/Nat/Totient.lean,Mathlib/Data/Ordmap/Invariants.lean,Mathlib/Data/Ordmap/Ordset.lean,Mathlib/Data/ZMod/ValMinAbs.lean,Mathlib/FieldTheory/ChevalleyWarning.lean,Mathlib/GroupTheory/Perm/Cycle/Type.lean,Mathlib/MeasureTheory/Covering/Vitali.lean,Mathlib/MeasureTheory/Integral/CircleIntegral.lean,Mathlib/MeasureTheory/Measure/Decomposition/Lebesgue.lean,Mathlib/MeasureTheory/Measure/Hausdorff.lean,Mathlib/MeasureTheory/Measure/SeparableMeasure.lean,Mathlib/NumberTheory/Bertrand.lean,Mathlib/NumberTheory/DiophantineApproximation/Basic.lean,Mathlib/SetTheory/Ordinal/Arithmetic.lean,Mathlib/SetTheory/Ordinal/Exponential.lean,Mathlib/SetTheory/Ordinal/FixedPoint.lean,Mathlib/SetTheory/Ordinal/Principal.lean,Mathlib/Tactic/Bound.lean,Mathlib/Tactic/CancelDenoms/Core.lean,Mathlib/Topology/Algebra/Monoid.lean,Mathlib/Topology/MetricSpace/Contracting.lean,Mathlib/Topology/MetricSpace/Dilation.lean,Mathlib/Topology/MetricSpace/Lipschitz.lean |
44 |
5 |
['JovanGerb', 'YaelDillies', 'github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
1-55177 1 day ago |
1-61900 1 day ago |
8-74244 8 days |
29275 |
wwylele author:wwylele |
feat(GroupTheory): add DivisibleHull |
This is part of Hahn embedding theorem #27268, where an a ordered group is first embedded in a divisible group / Q-module. I am aware at #25662 there is also an ongoing rewrite of `LocalizedModule` that this PR uses. Hopefully I avoided interfering it by using mostly with public API.
---
- [x] depends on: #29277
- [x] depends on: #29388
- [x] depends on: #29386
[](https://gitpod.io/from-referrer/)
|
t-group-theory |
485/0 |
Mathlib.lean,Mathlib/GroupTheory/DivisibleHull.lean |
2 |
51 |
['github-actions', 'mathlib4-dependent-issues-bot', 'vihdzp', 'wwylele'] |
nobody |
1-54598 1 day ago |
1-54598 1 day ago |
5-15776 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'] |
loefflerd and mariainesdff assignee:loefflerd assignee:mariainesdff |
1-52831 1 day ago |
80-55936 2 months ago |
80-55979 80 days |
29551 |
chrisflav author:chrisflav |
feat(CategoryTheory/Sites): the category of `1`-hypercovers up to homotopy |
We define the category of `1`-hypercovers up to homotopy as the category of `1`-hypercovers where morphisms are considered up to existence of a homotopy. We show that this category is cofiltered if the base category has pullbacks.
This category will be used to define a second construction of sheafification by taking certain colimits of multiequalizers over this category.
---
- [x] depends on: #29553
[](https://gitpod.io/from-referrer/)
|
large-import
t-category-theory
|
304/4 |
Mathlib/CategoryTheory/Sites/Coverage.lean,Mathlib/CategoryTheory/Sites/Hypercover/Homotopy.lean,Mathlib/CategoryTheory/Sites/Hypercover/One.lean,Mathlib/CategoryTheory/Sites/Hypercover/Zero.lean,Mathlib/CategoryTheory/Sites/Sieves.lean |
5 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
1-52038 1 day ago |
1-54114 1 day ago |
1-58045 1 day |
26039 |
tsuki8 author:tsuki8 |
feat(RingTheory/MvPolynomial/MonomialOrder): leadingTerm |
define the leadingTerm and prove some lemmas related to the def
`leadingTerm`: the leading term of `f` for the monomial ordering `m`
some basic lemmas about leadingTerm including:
1. `leadingTerm_eq_zero_iff`
2. `leadingTerm_image_sdiff_singleton_zero`
3. `leadingTerm_image_insert_zero`
4. `leadingTerm_zero`
5. `leadingTerm_degree_eq`
6. `leadingTerm_degree_eq'`
some lemmas about the degree of `f - m.leadingTerm f`:
1. `degree_sub_leadingTerm`
2. `degree_sub_leadingTerm_lt_degree`
3. `degree_sub_leadingTerm_lt_iff`
Co-authored-by: Junyu Guo @Hagb
---
- [ ] depends on: #24361
- [ ] depends on: #26148
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
new-contributor
awaiting-author
|
99/1 |
Mathlib/RingTheory/MvPolynomial/MonomialOrder.lean |
1 |
20 |
['Hagb', 'chrisflav', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
chrisflav assignee:chrisflav |
1-50910 1 day ago |
1-50910 1 day ago |
12-45707 12 days |
29227 |
robertmaxton42 author:robertmaxton42 |
feat (Limits.FunctorCategory): limitIsoFlipCompLim and colimitIsoFlipCompColim are natural |
Add `limIsoFlipCompWhiskerLim`, `limCompFlipIsoWhiskerLim`, `colimIsoFlipCompWhiskerColim`, `colimCompFlipIsoWhiskerColim`, each witnessing that their corresponding families of isomorphisms are natural in the diagram $F# .
---
Manually migrated from https://github.com/leanprover-community/mathlib4/pull/23992
[](https://gitpod.io/from-referrer/)
|
t-category-theory |
41/1 |
Mathlib/CategoryTheory/Limits/FunctorCategory/Basic.lean |
1 |
9 |
['github-actions', 'robertmaxton42', 'robin-carlier'] |
nobody |
1-50768 1 day ago |
1-50790 1 day ago |
7-73539 7 days |
28582 |
Thmoas-Guan author:Thmoas-Guan |
feat(Data): some lemmas about WithBot ENat |
Add some lemma about withBot ENat discovered when dealing with `ringKrullDim`
---
[](https://gitpod.io/from-referrer/)
|
t-data
awaiting-author
|
18/0 |
Mathlib/Data/ENat/Basic.lean |
1 |
4 |
['Ruben-VandeVelde', 'github-actions'] |
nobody |
1-47956 1 day ago |
1-47956 1 day ago |
24-63895 24 days |
19872 |
YaelDillies author:YaelDillies |
chore(GroupTheory/Index): rename `relindex` to `relIndex` |
Zulip discussion about renaming: [#PR reviews > #19872 rename relindex to relIndex @ 💬](https://leanprover.zulipchat.com/#narrow/channel/144837-PR-reviews/topic/.2319872.20rename.20relindex.20to.20relIndex/near/515908054)
---
- [x] depends on: #24044
[](https://gitpod.io/from-referrer/)
|
FLT
maintainer-merge
t-algebra
label:t-algebra$ |
297/191 |
Mathlib/Algebra/Module/ZLattice/Covolume.lean,Mathlib/FieldTheory/Relrank.lean,Mathlib/GroupTheory/Commensurable.lean,Mathlib/GroupTheory/CosetCover.lean,Mathlib/GroupTheory/GroupAction/Blocks.lean,Mathlib/GroupTheory/Index.lean,Mathlib/GroupTheory/IndexNormal.lean,Mathlib/GroupTheory/PGroup.lean,Mathlib/GroupTheory/Schreier.lean,Mathlib/GroupTheory/SchurZassenhaus.lean,Mathlib/GroupTheory/Sylow.lean,Mathlib/GroupTheory/Transfer.lean,Mathlib/LinearAlgebra/FreeModule/Finite/CardQuotient.lean,Mathlib/NumberTheory/ModularForms/CongruenceSubgroups.lean,Mathlib/NumberTheory/NumberField/Discriminant/Different.lean,Mathlib/NumberTheory/NumberField/Units/Regulator.lean,Mathlib/RingTheory/Ideal/Quotient/Index.lean |
17 |
29 |
['Ruben-VandeVelde', 'TwoFX', 'YaelDillies', 'alreadydone', 'eric-wieser', 'github-actions', 'joelriou', 'kbuzzard', 'leanprover-community-bot-assistant', 'loefflerd', 'madvorak', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'tb65536'] |
joelriou assignee:joelriou |
1-47158 1 day ago |
10-11188 10 days ago |
223-86035 223 days |
29278 |
Jlh18 author:Jlh18 |
feat: groupoid instance on quotient category |
Show that `CategoryTheory.Quotient` constructs a groupoid when the original category was a groupoid.
---
[](https://gitpod.io/from-referrer/)
|
large-import
new-contributor
t-category-theory
|
30/0 |
Mathlib/CategoryTheory/Quotient.lean |
1 |
4 |
['Jlh18', 'github-actions', 'joelriou'] |
riccardobrasca assignee:riccardobrasca |
1-46963 1 day ago |
1-46966 1 day ago |
9-80393 9 days |
27849 |
robin-carlier author:robin-carlier |
feat(CategoryTheory/Bicategory/Functor): strictly unitary lax/pseudo functors |
We define strictly unitary lax/pseudo functors between bicategories. A lax (resp. pseudo-)functor from `C` to `D` is strictly unitary if `F.map(𝟙 X) = 𝟙 (F.obj X)` and if the 2-cell `mapId` is the identity 2-cell induced by this equality. We provide a constructor for those that do not require the `mapId` field.
Although this structure is somewhat "evil" from a purely categorical perspective (it mentions non-definitonal equality of objects in a 1-category), these class of functors are of interest: strictly unitary lax functors are part of the definition of the Duskin nerve of a bicategory (which embeds bicategories in the theory of simplicial sets), while strictly unitary pseudofunctors are part of the definition of the 2-nerve of a bicategory, which embeds bicategories into the theory of simplicial categories.
This PR is part of an ongoing work that will hopefully culminate with the construction of the Duskin Nerve, as well as a proof of the fact that the Duskin nerve of a locally groupoidal bicategory is a quasicategory.
---
Two designs were possible here: making `StrictlyUnitary` a class on lax/pseudo-functors to state that some functors/constructions are strictly unitary, or bundling it as a structure on its own.
Since my plan for the follow-up PRs is to use the type of strictly lax unitary functors between some bicategories (e.g to define lax-composable arrows in a bicategory `C`, which will be by definition `StrictlyUnitaryLaxFunctor (LocallyDiscrete (Fin n)) C`), I chose to bundle them directly, to avoid an extra layer when working with the type of those objects.
I did include strict associativity for strictly unitary lax functors but not for pseudofunctors. The reason is that the Duskin nerve mentions the 1-category of bicategories and strictly unitary lax functors (hence, this strict associativity/unitality), but the 2-nerve mentions the bicategory of bicategories, strictly unitary pseudofunctors and "icons" (identity-component oplax natural transformations): the statement for associativity for pseudofunctors will wait for icons, and will probably not be stated as an equality of pseudofunctors.
[](https://gitpod.io/from-referrer/)
|
t-category-theory
ready-to-merge
delegated
|
356/0 |
Mathlib.lean,Mathlib/CategoryTheory/Bicategory/Functor/StrictlyUnitary.lean |
2 |
8 |
['adamtopaz', 'github-actions', 'mathlib-bors', 'robin-carlier'] |
adamtopaz assignee:adamtopaz |
1-45164 1 day ago |
1-47145 1 day ago |
38-25023 38 days |
29569 |
chrisflav author:chrisflav |
chore(RingTheory/LocalProperties): add algebra versions of exactness lemmas |
The module variants are less convenient to apply directly in the case of algebras.
From Pi1.
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory |
67/0 |
Mathlib/RingTheory/LocalProperties/Exactness.lean |
1 |
1 |
['github-actions'] |
nobody |
1-41219 1 day ago |
1-41219 1 day ago |
1-41342 1 day |
29570 |
eric-wieser author:eric-wieser |
fix: substitute infotrees in linters |
I don't know whether this is necessary in these particular cases, but I've seen places where it is.
There are a handful more of these cases in Batteries.
---
[](https://gitpod.io/from-referrer/)
|
|
2/2 |
Mathlib/Tactic/Linter/Style.lean,Mathlib/Tactic/TacticAnalysis.lean |
2 |
1 |
['github-actions'] |
nobody |
1-40321 1 day ago |
1-40387 1 day ago |
0-0 0 seconds |
29468 |
kim-em author:kim-em |
feat: add `cutsat` and `grobner` macro frontends to `grind` |
These macros will be replaced with proper implementations in Lean soon,
but are starting out here for quick experimentation.
Notes:
* I'll later replace these with an implementation that uses a minimal configuration
and then reactivates modules as needed.
* It would be nice if these macros supported all the `grind` configurations, too. |
|
200/2 |
Archive/Imo/Imo1994Q1.lean,Mathlib.lean,Mathlib/RingTheory/ClassGroup.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Common.lean,Mathlib/Tactic/Grind.lean,MathlibTest/grind/grobner.lean |
7 |
7 |
['eric-wieser', 'euprunin', 'github-actions', 'hrmacbeth', 'kim-em'] |
nobody |
1-39269 1 day ago |
3-81248 3 days ago |
3-81229 3 days |
29493 |
kim-em author:kim-em |
chore: grind golf in Mathlib.Logic |
More golfs identified by `linter.tacticAnalysis.terminalToGrind`. |
maintainer-merge
t-logic
|
8/20 |
Mathlib/Logic/Basic.lean,Mathlib/Logic/Function/Basic.lean,Mathlib/Logic/Relation.lean,scripts/noshake.json |
4 |
6 |
['euprunin', 'github-actions', 'grunweg', 'kim-em'] |
nobody |
1-39173 1 day ago |
3-6486 3 days ago |
3-15297 3 days |
29573 |
kim-em author:kim-em |
chore: deprecate `Traversable` deriving handler |
This broke on `nightly-testing`. It's very probably fixable, but I'm not interested in doing that myself, and I think this is a good opportunity to remove some code which has not been used since 2018. |
file-removed |
7/3 |
Mathlib.lean,Mathlib/Deprecated/Tactic/DeriveTraversable.lean,Mathlib/Tactic.lean,MathlibTest/Traversable.lean |
4 |
1 |
['github-actions'] |
nobody |
1-35911 1 day ago |
1-35911 1 day ago |
1-36001 1 day |
26129 |
LessnessRandomness author:LessnessRandomness |
feat(Geometry/Euclidean/Angle/Unoriented): triangle inequality for angles |
This PR continues the work from #24206.
Original PR: https://github.com/leanprover-community/mathlib4/pull/24206 |
new-contributor
t-euclidean-geometry
|
223/11 |
Mathlib.lean,Mathlib/Analysis/InnerProductSpace/Basic.lean,Mathlib/Geometry/Euclidean/Angle/Unoriented/Affine.lean,Mathlib/Geometry/Euclidean/Angle/Unoriented/Basic.lean,Mathlib/Geometry/Euclidean/Angle/Unoriented/TriangleInequality.lean |
5 |
36 |
['JovanGerb', 'LessnessRandomness', 'Timeroot', 'github-actions', 'jsm28', 'mathlib4-merge-conflict-bot'] |
jsm28 assignee:jsm28 |
1-34925 1 day ago |
8-39657 8 days ago |
83-67453 83 days |
27956 |
bryangingechen author:bryangingechen |
feat: automation for removing outdated deprecations |
This is a new weekly workflow that opens a PR attempting to remove deprecated aliases / declarations older than 6 months and then sends a Zulip message to the `nightly-testing` channel. It also supports being triggered manually with a custom date as well as a "dry-run" mode, which only prints the edits that would be done without actually doing them.
cf. [#mathlib reviewers > auto-removing oudated deprecations @ 💬](https://leanprover.zulipchat.com/#narrow/channel/345428-mathlib-reviewers/topic/auto-removing.20oudated.20deprecations/near/532535945)
The workflow and shell script are adapted from `nolints.yml` and `scripts/update_nolints_CI.sh`, respectively.
The python script was mostly written by Claude, though I did check it. The regex is adapted from ones used in #21271 by YaelDillies and #29287 by kim-em.
---
See #29336 for an example of the changes generated by the script. |
CI |
330/0 |
.github/workflows/remove_deprecated_decls.yml,scripts/README.md,scripts/remove_deprecated_decls.py,scripts/remove_deprecated_decls_CI.sh |
4 |
2 |
['bryangingechen', 'github-actions'] |
robertylewis assignee:robertylewis |
1-34923 1 day ago |
9-33043 9 days ago |
39-34110 39 days |
28571 |
euprunin author:euprunin |
chore(RingTheory): golf entire `mem_extended_iff`, `coeff_opRingEquiv` and `comp_assoc` using `rfl` |
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory |
4/12 |
Mathlib/RingTheory/ClassGroup.lean,Mathlib/RingTheory/FractionalIdeal/Extended.lean,Mathlib/RingTheory/Polynomial/Opposites.lean,Mathlib/RingTheory/PolynomialLaw/Basic.lean |
4 |
7 |
['euprunin', 'github-actions', 'grunweg', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'mathlib4-merge-conflict-bot'] |
chrisflav assignee:chrisflav |
1-34920 1 day ago |
8-45735 8 days ago |
18-19370 18 days |
28981 |
euprunin author:euprunin |
chore(AlgebraicTopology/ModelCategory): remove redundant `have` in `mk'.cm3a_aux` |
---
[](https://gitpod.io/from-referrer/)
|
t-algebraic-topology |
0/1 |
Mathlib/AlgebraicTopology/ModelCategory/Basic.lean |
1 |
6 |
['euprunin', 'github-actions', 'grunweg', 'leanprover-bot', 'leanprover-community-mathlib4-bot'] |
robin-carlier assignee:robin-carlier |
1-34918 1 day ago |
8-52301 8 days ago |
8-59147 8 days |
29223 |
dwrensha author:dwrensha |
feat: norm_num extension for abs |
Adds a `norm_num` extension for the [absolute value operator](https://github.com/leanprover-community/mathlib4/blob/3a941a8fd0acf2b70463b31aeb8ce08bb214a512/Mathlib/Algebra/Order/Group/Unbundled/Abs.lean#L39-L40).
---
[](https://gitpod.io/from-referrer/)
|
t-meta |
93/5 |
Mathlib.lean,Mathlib/Analysis/Complex/ExponentialBounds.lean,Mathlib/Tactic.lean,Mathlib/Tactic/NormNum.lean,Mathlib/Tactic/NormNum/Abs.lean,MathlibTest/norm_num_abs.lean |
6 |
17 |
['dwrensha', 'eric-wieser', 'github-actions', 'plp127', 'vihdzp'] |
adamtopaz assignee:adamtopaz |
1-34916 1 day ago |
8-67956 8 days ago |
10-44495 10 days |
29270 |
euprunin author:euprunin |
chore: remove redundant `refine` invocations |
---
**Note:** Although technically redundant, some of these may be worth keeping for readability, or other reasons. Let me know if you think any should stay.
---
[](https://gitpod.io/from-referrer/)
|
|
4/12 |
Mathlib/Algebra/Order/GroupWithZero/Lex.lean,Mathlib/Algebra/Polynomial/Smeval.lean,Mathlib/AlgebraicGeometry/Limits.lean,Mathlib/Geometry/Manifold/LocalInvariantProperties.lean,Mathlib/Probability/Density.lean |
5 |
4 |
['github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot'] |
dupuisf assignee:dupuisf |
1-34915 1 day ago |
10-40060 10 days ago |
10-43439 10 days |
29250 |
Jlh18 author:Jlh18 |
chore: rename hom_to_functor, id_to_functor |
The files `CategoryTheory.Category.Grpd` and `CategoryTheory.Category.Cat` should be consistent in naming conventions and style. Here I renamed `CategoryTheory.Grpd.hom_to_functor` to `CategoryTheory.Grpd.comp_eq_comp` to mirror `CategoryTheory.Cat.comp_eq_comp`. Similarly I renamed `CategoryTheory.Grpd.id_to_functor` to `CategoryTheory.Grpd.id_eq_eq`
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-category-theory
easy
|
9/3 |
Mathlib/AlgebraicTopology/FundamentalGroupoid/InducedMaps.lean,Mathlib/CategoryTheory/Category/Grpd.lean |
2 |
4 |
['Jlh18', 'github-actions', 'joelriou'] |
robin-carlier assignee:robin-carlier |
1-34915 1 day ago |
8-75620 8 days ago |
10-74567 10 days |
29301 |
harahu author:harahu |
doc: hyphenate attributive compound adjectives ending in "preserving" |
Compound adjectives that are attributive (coming before their noun) should almost always be hyphenated in English.
This PR covers such adjectives that are ending in "preserving".
---
[](https://gitpod.io/from-referrer/)
|
|
71/71 |
Mathlib/Algebra/Order/CompleteField.lean,Mathlib/AlgebraicTopology/SimplicialSet/Boundary.lean,Mathlib/CategoryTheory/Monoidal/Cartesian/Basic.lean,Mathlib/CategoryTheory/Monoidal/OfHasFiniteProducts.lean,Mathlib/CategoryTheory/Preadditive/LeftExact.lean,Mathlib/CategoryTheory/Sites/Coherent/ExtensiveSheaves.lean,Mathlib/CategoryTheory/Sites/PreservesLocallyBijective.lean,Mathlib/CategoryTheory/Sites/Sheafification.lean,Mathlib/Condensed/Discrete/Colimit.lean,Mathlib/Condensed/Discrete/LocallyConstant.lean,Mathlib/Dynamics/BirkhoffSum/QuasiMeasurePreserving.lean,Mathlib/Dynamics/Circle/RotationNumber/TranslationNumber.lean,Mathlib/Dynamics/Ergodic/Ergodic.lean,Mathlib/Dynamics/Ergodic/MeasurePreserving.lean,Mathlib/GroupTheory/GroupAction/DomAct/Basic.lean,Mathlib/GroupTheory/SpecificGroups/KleinFour.lean,Mathlib/LinearAlgebra/Reflection.lean,Mathlib/MeasureTheory/Constructions/Pi.lean,Mathlib/MeasureTheory/Function/AEEqFun.lean,Mathlib/MeasureTheory/Function/LpSpace/Basic.lean,Mathlib/MeasureTheory/Function/LpSpace/ContinuousCompMeasurePreserving.lean,Mathlib/MeasureTheory/Function/LpSpace/DomAct/Continuous.lean,Mathlib/MeasureTheory/Group/AEStabilizer.lean,Mathlib/MeasureTheory/Group/Action.lean,Mathlib/MeasureTheory/Group/FundamentalDomain.lean,Mathlib/MeasureTheory/Measure/ContinuousPreimage.lean,Mathlib/MeasureTheory/Measure/Prod.lean,Mathlib/MeasureTheory/Measure/QuasiMeasurePreserving.lean,Mathlib/MeasureTheory/Measure/Restrict.lean,Mathlib/Probability/Density.lean,Mathlib/RingTheory/FractionalIdeal/Norm.lean,Mathlib/RingTheory/GradedAlgebra/HomogeneousLocalization.lean,Mathlib/RingTheory/OrderOfVanishing.lean,Mathlib/Topology/Sheaves/SheafCondition/Sites.lean,Mathlib/Topology/Sheaves/SheafOfFunctions.lean |
35 |
2 |
['github-actions', 'harahu'] |
robin-carlier assignee:robin-carlier |
1-34912 1 day ago |
10-4291 10 days ago |
10-4272 10 days |
29316 |
euprunin author:euprunin |
chore: remove redundant `suffices` invocations |
---
**Note:** Although technically redundant, some of these may be worth keeping for readability, or other reasons. Let me know if you think any should stay.
---
[](https://gitpod.io/from-referrer/)
|
|
0/4 |
Mathlib/Algebra/ContinuedFractions/Computation/Approximations.lean,Mathlib/Algebra/ContinuedFractions/Determinant.lean,Mathlib/MeasureTheory/Function/LpSeminorm/Basic.lean |
3 |
4 |
['github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot'] |
tb65536 assignee:tb65536 |
1-34911 1 day ago |
9-69370 9 days ago |
9-75381 9 days |
29317 |
euprunin author:euprunin |
chore: remove redundant `generalize`, `induction`, `repeat'` and `unfold` invocations |
---
**Note:** Although technically redundant, some of these may be worth keeping for readability, or other reasons. Let me know if you think any should stay.
---
[](https://gitpod.io/from-referrer/)
|
|
3/12 |
Mathlib/Algebra/Order/Archimedean/Class.lean,Mathlib/Data/ENNReal/Real.lean,Mathlib/NumberTheory/LSeries/HurwitzZetaOdd.lean,Mathlib/RingTheory/Polynomial/Opposites.lean |
4 |
7 |
['JovanGerb', 'euprunin', 'github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot'] |
robin-carlier assignee:robin-carlier |
1-34910 1 day ago |
9-62861 9 days ago |
9-75060 9 days |
29344 |
JovanGerb author:JovanGerb |
feat(Geometry/Euclidean/Sphere/Power): use side condition `p ∈ line[ℝ, a, b]` |
This PR changes the side condition used in theorems about `Sphere.power` to be `p ∈ line[ℝ, a, b]`. This is symmetric in `a` and `b`, and more general that the current condition.
TODO (in this PR?): add some basic lemmas about `p ∈ line[ℝ, a, b]`.
TODO (in another PR): prove the power theorems about `Sphere.secondInter`, which is more general in the sense that it also includes the case where `a` and `b` coincide, and then `p` is on the tangent line.
---
[](https://gitpod.io/from-referrer/)
|
t-euclidean-geometry |
31/34 |
Mathlib/Geometry/Euclidean/Sphere/Power.lean |
1 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
jsm28 assignee:jsm28 |
1-34908 1 day ago |
8-39702 8 days ago |
8-56608 8 days |
29559 |
j-loreaux author:j-loreaux |
feat: add C⋆-algebra instances for elemental algebras |
---
[](https://gitpod.io/from-referrer/)
|
t-analysis
delegated
|
21/2 |
Mathlib/Analysis/CStarAlgebra/Classes.lean,Mathlib/Topology/Algebra/StarSubalgebra.lean |
2 |
4 |
['eric-wieser', 'github-actions', 'mathlib-bors'] |
nobody |
1-34338 1 day ago |
1-34338 1 day ago |
0-36932 10 hours |
29574 |
JarodUW author:JarodUW |
Regular local rings are domains |
We have added three new files in Mathlib/RingTheory/LocalRing
* EmbeddingDimension.lean
* LocalRingDimension.lean
* RegularLocalRings.lean
We have added two lemmas and an instance in Mathlib/RingTheory/LocalRing/RingHom/Basic.lean
This work was done by Jarod Alper and Brian Nugent.
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
new-contributor
|
905/1 |
Mathlib/RingTheory/LocalRing/EmbeddingDimension.lean,Mathlib/RingTheory/LocalRing/LocalRingDimension.lean,Mathlib/RingTheory/LocalRing/RegularLocalRings.lean,Mathlib/RingTheory/LocalRing/RingHom/Basic.lean |
4 |
1 |
['github-actions'] |
nobody |
1-33820 1 day ago |
1-33826 1 day ago |
1-33870 1 day |
28706 |
euprunin author:euprunin |
chore: golf entire `dite_ne_left_iff`, `exists_prime_lt_and_le_two_mul_succ`, `lt_up` and `sUnion_mem_empty_univ` using `grind` |
---
[](https://gitpod.io/from-referrer/)
|
maintainer-merge |
4/12 |
Mathlib/Data/Set/Lattice.lean,Mathlib/Logic/Basic.lean,Mathlib/NumberTheory/Bertrand.lean,Mathlib/RingTheory/NoetherNormalization.lean |
4 |
9 |
['euprunin', 'github-actions', 'grunweg', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'mathlib4-merge-conflict-bot', 'tb65536'] |
tb65536 assignee:tb65536 |
1-33816 1 day ago |
1-33816 1 day ago |
15-10955 15 days |
29453 |
kim-em author:kim-em |
chore: grind annotations in Data/Bool |
|
t-data |
40/46 |
Mathlib/Data/Bool/Basic.lean,Mathlib/Data/Bool/Count.lean,Mathlib/Data/Bool/Set.lean |
3 |
1 |
['github-actions'] |
nobody |
1-30484 1 day ago |
4-37210 4 days ago |
4-37256 4 days |
27307 |
xyzw12345 author:xyzw12345 |
feat(RingTheory/GradedAlgebra): homogeneous relation |
This PR continues the work from #22279.
Original PR: https://github.com/leanprover-community/mathlib4/pull/22279 |
t-ring-theory |
391/0 |
Mathlib.lean,Mathlib/Algebra/Algebra/Equiv.lean,Mathlib/Algebra/DirectSum/Basic.lean,Mathlib/Algebra/DirectSum/Module.lean,Mathlib/Algebra/Module/LinearMap/Defs.lean,Mathlib/Algebra/Ring/Equiv.lean,Mathlib/Algebra/RingQuot.lean,Mathlib/RingTheory/GradedAlgebra/Basic.lean,Mathlib/RingTheory/GradedAlgebra/HomogeneousRelation.lean |
9 |
7 |
['chrisflav', 'eric-wieser', 'github-actions', 'xyzw12345'] |
ocfnash assignee:ocfnash |
1-22893 1 day ago |
39-61300 1 month ago |
54-72620 54 days |
29004 |
euprunin author:euprunin |
WIP: experiment: bench `:= rfl` vs `:= by rfl` |
---
[](https://gitpod.io/from-referrer/)
|
WIP |
141/248 |
Mathlib/Algebra/Algebra/NonUnitalHom.lean,Mathlib/Algebra/Category/ModuleCat/Presheaf.lean,Mathlib/Algebra/DirectSum/Module.lean,Mathlib/Algebra/DirectSum/Ring.lean,Mathlib/Algebra/Group/AddChar.lean,Mathlib/Algebra/Group/Subgroup/Defs.lean,Mathlib/Algebra/GroupWithZero/ProdHom.lean,Mathlib/Algebra/Homology/HomotopyCategory/HomComplex.lean,Mathlib/Algebra/Homology/ShortComplex/LeftHomology.lean,Mathlib/Algebra/Homology/Single.lean,Mathlib/Algebra/Lie/Basic.lean,Mathlib/Algebra/Lie/OfAssociative.lean,Mathlib/Algebra/Lie/Submodule.lean,Mathlib/Algebra/Order/Hom/MonoidWithZero.lean,Mathlib/Algebra/Order/Hom/Ring.lean,Mathlib/Algebra/Polynomial/AlgebraMap.lean,Mathlib/Algebra/Polynomial/Derivation.lean,Mathlib/Algebra/Polynomial/Module/Basic.lean,Mathlib/Algebra/Ring/Hom/Defs.lean,Mathlib/Algebra/RingQuot.lean,Mathlib/Algebra/Vertex/HVertexOperator.lean,Mathlib/Algebra/Vertex/VertexOperator.lean,Mathlib/AlgebraicTopology/SimplicialSet/StdSimplex.lean,Mathlib/Analysis/Asymptotics/ExpGrowth.lean,Mathlib/Analysis/CStarAlgebra/GelfandDuality.lean,Mathlib/Analysis/Calculus/FDeriv/Prod.lean,Mathlib/Analysis/Complex/UpperHalfPlane/Basic.lean,Mathlib/Analysis/Distribution/SchwartzSpace.lean,Mathlib/Analysis/Normed/Affine/Isometry.lean,Mathlib/Analysis/Normed/Group/Seminorm.lean,Mathlib/Analysis/Normed/Module/Span.lean,Mathlib/Analysis/SpecialFunctions/Complex/CircleAddChar.lean,Mathlib/Analysis/SpecialFunctions/Stirling.lean,Mathlib/CategoryTheory/Closed/Monoidal.lean,Mathlib/CategoryTheory/Distributive/Monoidal.lean,Mathlib/CategoryTheory/Limits/Presheaf.lean,Mathlib/CategoryTheory/Limits/Shapes/Pullback/Cospan.lean,Mathlib/CategoryTheory/Monoidal/Comon_.lean,Mathlib/CategoryTheory/Monoidal/Mod_.lean,Mathlib/CategoryTheory/Monoidal/Mon_.lean,Mathlib/CategoryTheory/Shift/ShiftedHomOpposite.lean,Mathlib/CategoryTheory/Yoneda.lean,Mathlib/Combinatorics/SimpleGraph/Walk.lean,Mathlib/Computability/AkraBazzi/AkraBazzi.lean,Mathlib/Computability/AkraBazzi/SumTransform.lean,Mathlib/Data/Matrix/Basic.lean,Mathlib/Data/Nat/Factorization/PrimePow.lean,Mathlib/Data/Nat/PartENat.lean,Mathlib/Data/PFunctor/Multivariate/Basic.lean,Mathlib/Data/Real/Embedding.lean,Mathlib/Data/Rel.lean,Mathlib/Data/Seq/Basic.lean,Mathlib/Data/Set/Lattice.lean,Mathlib/Data/Set/Pairwise/Lattice.lean,Mathlib/Data/Subtype.lean,Mathlib/Geometry/Manifold/Bordism.lean,Mathlib/GroupTheory/Coxeter/Basic.lean,Mathlib/GroupTheory/GroupAction/Hom.lean,Mathlib/GroupTheory/SpecificGroups/Quaternion.lean,Mathlib/LinearAlgebra/AffineSpace/Simplex/Basic.lean,Mathlib/LinearAlgebra/Dual/Defs.lean,Mathlib/LinearAlgebra/Lagrange.lean,Mathlib/LinearAlgebra/Matrix/GeneralLinearGroup/Defs.lean,Mathlib/LinearAlgebra/Multilinear/TensorProduct.lean,Mathlib/LinearAlgebra/Projectivization/Action.lean,Mathlib/LinearAlgebra/RootSystem/Hom.lean,Mathlib/LinearAlgebra/RootSystem/Reduced.lean,Mathlib/LinearAlgebra/Span/Basic.lean,Mathlib/LinearAlgebra/TensorProduct/Pi.lean,Mathlib/MeasureTheory/MeasurableSpace/Embedding.lean,Mathlib/ModelTheory/Semantics.lean,Mathlib/NumberTheory/FLT/Polynomial.lean,Mathlib/NumberTheory/FactorisationProperties.lean,Mathlib/NumberTheory/Harmonic/ZetaAsymp.lean,Mathlib/NumberTheory/Padics/WithVal.lean,Mathlib/Order/BoundedOrder/Basic.lean,Mathlib/RepresentationTheory/Coinvariants.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/Functoriality.lean,Mathlib/RepresentationTheory/Homological/GroupHomology/LowDegree.lean,Mathlib/RingTheory/AlgebraTower.lean,Mathlib/RingTheory/Bialgebra/Hom.lean,Mathlib/RingTheory/HahnSeries/Addition.lean,Mathlib/RingTheory/Ideal/Norm/AbsNorm.lean,Mathlib/RingTheory/Ideal/Quotient/Operations.lean,Mathlib/SetTheory/Surreal/Basic.lean,Mathlib/SetTheory/ZFC/Class.lean,Mathlib/Tactic/Module.lean,Mathlib/Tactic/NormNum/PowMod.lean,Mathlib/Topology/Algebra/Algebra/Equiv.lean,Mathlib/Topology/Algebra/Module/WeakDual.lean,Mathlib/Topology/Category/Profinite/Nobeling/Basic.lean,Mathlib/Topology/Category/Profinite/Nobeling/ZeroLimit.lean,Mathlib/Topology/Category/TopCat/Opens.lean,Mathlib/Topology/ContinuousMap/Units.lean,Mathlib/Topology/LocallyFinsupp.lean,Mathlib/Topology/PartitionOfUnity.lean,Mathlib/Topology/Sets/Closeds.lean |
97 |
16 |
['eric-wieser', 'euprunin', 'github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot'] |
nobody |
1-20728 1 day ago |
1-60550 1 day ago |
0-84080 23 hours |
29576 |
kim-em author:kim-em |
chore: add grind annotations for homomorphisms |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
7/7 |
Mathlib/Algebra/Group/Hom/Defs.lean |
1 |
1 |
['github-actions'] |
nobody |
1-20463 1 day ago |
1-20477 1 day ago |
0-0 0 seconds |
29136 |
YaelDillies author:YaelDillies |
feat(CategoryTheory/Monoidal): `mapMon` of a lax-braided functor is lax-braided |
Also move the `BraidedCategory (Mon_ C)` instance earlier in the file to avoid splitting up the functor material. I think it makes more sense like this (defining `Mon_Class`, then `Mon_`, then `Functor.mapMon`).
From Toric
---
[](https://gitpod.io/from-referrer/)
|
toric
t-category-theory
|
431/399 |
Mathlib/Algebra/Category/CoalgCat/ComonEquivalence.lean,Mathlib/CategoryTheory/Monoidal/Mon_.lean |
2 |
3 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
TwoFX assignee:TwoFX |
1-13875 1 day ago |
1-13897 1 day ago |
13-3605 13 days |
29577 |
kim-em author:kim-em |
feat: alternating series error bound |
Thanks for the hints from @sgouezel at [#Is there code for X? > error term for summable alternating series?](https://leanprover.zulipchat.com/#narrow/channel/217875-Is-there-code-for-X.3F/topic/error.20term.20for.20summable.20alternating.20series.3F/with/538984368). |
|
39/0 |
Mathlib/Analysis/SpecificLimits/Normed.lean,Mathlib/Topology/Algebra/InfiniteSum/Order.lean |
2 |
2 |
['github-actions', 'loefflerd'] |
nobody |
1-7641 1 day ago |
1-19378 1 day ago |
1-19359 1 day |
29548 |
Parcly-Taxel author:Parcly-Taxel |
feat: add `induction'` to the deprecated syntax linter |
Exactly like `cases'`.
---
* [x] depends on: #29542 |
awaiting-zulip
tech debt
t-linter
|
41/2 |
Mathlib/Init.lean,Mathlib/Tactic/Linter/DeprecatedSyntaxLinter.lean,MathlibTest/DeprecatedSyntaxLinter.lean |
3 |
3 |
['Parcly-Taxel', 'github-actions', 'grunweg'] |
grunweg assignee:grunweg |
1-5652 1 day ago |
1-5652 1 day ago |
0-83159 23 hours |
26096 |
vasnesterov author:vasnesterov |
feat(Topology/Instances): Cantor set is the set of ternary numbers without `1`s |
* Prove `zero_two_sequence_ofDigits_mem_cantorSet`: If `x = 0.d₀d₁...` in base-3, and none of the digits `dᵢ` is `1`, then `x` belongs to the Cantor set.
* Prove `zero_two_sequence_ofDigits_unique`: such a representation is uniquie.
* Define `toTernary` which converts a real number from the Cantor set to its ternary representation without `1`s.
* Prove `ofDigits_cantorToTernary : ofDigits (cantorToTernary x) = x`.
---
This is a prerequisite for #26136.
- [x] depends on: #26001
- [x] depends on: #26021
[](https://gitpod.io/from-referrer/)
|
large-import
t-topology
|
231/0 |
Mathlib/Topology/Instances/CantorSet.lean,scripts/noshake.json |
2 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
1-5138 1 day ago |
1-47450 1 day ago |
1-47811 1 day |
29445 |
j-loreaux author:j-loreaux |
chore(Analysis/NormedSpace/Extend): split file |
This PR accomplishes a few tasks:
1. splits the file according to whether the material needs the operator norm on continuous linear map. This will help us avoid importing the operator norm into `LocallyConvex/` in an upcoming transition of material from `NormedSpace/HahnBanach/` into other folders.
2. moves the resulting files out of the `NormedSpace` folder in accordance with #28698.
3. Cleans up the declarations / proofs / docstrings a small amount.
4. Uses `Module.Dual` spelling for the linear maps.
This is part of #28698 to migrate the material in `Analysis/NormedSpace/` to other locations.
---
Although this PR does a few different jobs, it should be reviewable on a commit-by-commit basis relatively easily.
The first commit splits the file. In so doing it was necessary to change slightly a few things (e.g., `ContinuousLinearMap.extendTo𝕜'` no longer uses `LinearMap.mkContinuous` because we don't have access to the operator norm, but continuity is still trivially provable; but also, due to the reordering, we can make `ContinuousLinearMap.norm_extendTo𝕜'_bound` a statement directly about `fr.extendTo𝕜'` instead of `fr.toLinearMap.extenTo𝕜'`). I think this is uniformly better. Here we also correct the module documentation in minor ways.
The second commit minimizes imports and adds an `assert_not_exists` to make sure we don't import the operator norm too early.
The third commit cleans up a few proofs.
The fourth commit imports `Mathlib.LinearAlgebra.Dual.Defs` so that we can use the `Module.Dual` spelling. I checked that this is the only new file imported (including transitive imports), so it's a lightweight change.
Note that yet another task (which we reserve for a future PR because of the challenge for review) is to rename from `LinearMap.extendTo𝕜` to something more appropriate that doesn't mention notation, e.g., `Module.Dual.rclikeExtend`.
[](https://gitpod.io/from-referrer/)
|
file-removed
tech debt
t-analysis
awaiting-author
|
194/159 |
Mathlib.lean,Mathlib/Analysis/Normed/Module/RCLike/Extend.lean,Mathlib/Analysis/NormedSpace/Extend.lean,Mathlib/Analysis/NormedSpace/HahnBanach/Extension.lean,Mathlib/Analysis/NormedSpace/HahnBanach/Separation.lean,Mathlib/Analysis/RCLike/Extend.lean |
6 |
2 |
['faenuccio', 'github-actions', 'j-loreaux'] |
nobody |
0-83381 23 hours ago |
0-83381 23 hours ago |
3-59741 3 days |
29432 |
lecopivo author:lecopivo |
feat: `data_synth` tactic to prove `HasFDerivAt 𝕜 f ?f' x` and similar |
New tactic `data_synth` that can prove proposition with holes e.g. figure out what `?f'` is and prove `HasFDerivAt 𝕜 f ?f' x`
---
Tactic `data_synth` is designed to synthesize some data that satisfies some proposition. The canonical example is `HasFDerivAt 𝕜 f ?f' x`, this tactic will figure out `f'` and provide proof of `HasFDerivAt 𝕜 f f' x`.
Another examples: `HasBoundinbBall s ?center ?radius` or `IsPolynomial f ?p`
```
def HasBoundingBall (s : Set α) (center : α) (radius : ℝ) : Prop :=
s ⊆ Metric.closedBall center radius
def IsPolynomial (f : R → R) (p : Polynomial R) :=
f = p.eval
``` |
t-meta
WIP
|
1943/0 |
Mathlib/Tactic/DataSynth.lean,Mathlib/Tactic/DataSynth/Attr.lean,Mathlib/Tactic/DataSynth/Core.lean,Mathlib/Tactic/DataSynth/Decl.lean,Mathlib/Tactic/DataSynth/Elab.lean,Mathlib/Tactic/DataSynth/FDeriv.lean,Mathlib/Tactic/DataSynth/FDeriv/Basic.lean,Mathlib/Tactic/DataSynth/FDeriv/Dispatch.lean,Mathlib/Tactic/DataSynth/FDeriv/Init.lean,Mathlib/Tactic/DataSynth/FDeriv/Simproc.lean,Mathlib/Tactic/DataSynth/Tests/BoundingBall.lean,Mathlib/Tactic/DataSynth/Tests/Compilation.lean,Mathlib/Tactic/DataSynth/Tests/FDeriv.lean,Mathlib/Tactic/DataSynth/Tests/FDerivInit.lean,Mathlib/Tactic/DataSynth/Tests/FwdDeriv.lean,Mathlib/Tactic/DataSynth/Tests/Normalize.lean,Mathlib/Tactic/DataSynth/Tests/Polynomial.lean,Mathlib/Tactic/DataSynth/Theorems.lean,Mathlib/Tactic/DataSynth/ToBatteries.lean,Mathlib/Tactic/DataSynth/Types.lean |
20 |
1 |
['github-actions'] |
nobody |
0-83175 23 hours ago |
4-81230 4 days ago |
0-11559 3 hours |
25138 |
chrisflav author:chrisflav |
chore(RingTheory/Ideal): make `RingHom.ker` take a `RingHom` instead of `RingHomClass` |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
72/71 |
Mathlib/Algebra/Algebra/Hom.lean,Mathlib/Algebra/Algebra/Subalgebra/Operations.lean,Mathlib/Algebra/Polynomial/Module/AEval.lean,Mathlib/Combinatorics/Nullstellensatz.lean,Mathlib/LinearAlgebra/TensorProduct/RightExactness.lean,Mathlib/RingTheory/Algebraic/Basic.lean,Mathlib/RingTheory/FinitePresentation.lean,Mathlib/RingTheory/Ideal/Maps.lean,Mathlib/RingTheory/Ideal/Quotient/Operations.lean,Mathlib/RingTheory/Localization/Algebra.lean,Mathlib/RingTheory/Nilpotent/Lemmas.lean,Mathlib/RingTheory/NoetherNormalization.lean,Mathlib/RingTheory/Polynomial/Basic.lean,Mathlib/Topology/Algebra/Module/CharacterSpace.lean,Mathlib/Topology/ContinuousMap/Ideals.lean |
15 |
5 |
['chrisflav', 'erdOne', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant'] |
nobody |
0-83145 23 hours ago |
1-1195 1 day ago |
10-65674 10 days |
29310 |
Louddy author:Louddy |
feat(SkewMonoidAlgebra): algebra instance |
Algebra instance for skew monoid algebras.
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$ |
65/12 |
Mathlib/Algebra/SkewMonoidAlgebra/Basic.lean |
1 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
0-79041 21 hours ago |
0-79069 21 hours ago |
8-55899 8 days |
29589 |
grunweg author:grunweg |
feat: add mfderiv_prod and mfderiv_prodMap |
Part of my bordism theory project: these will be needed for https://github.com/leanprover-community/mathlib4/pull/22059.
Updated version of #22642.
---
[](https://gitpod.io/from-referrer/)
|
t-differential-geometry
WIP
|
142/79 |
Mathlib/Analysis/Calculus/FDeriv/Prod.lean,Mathlib/Geometry/Manifold/MFDeriv/Basic.lean,Mathlib/Geometry/Manifold/MFDeriv/SpecificFunctions.lean |
3 |
1 |
['github-actions'] |
nobody |
0-79019 21 hours ago |
0-79054 21 hours ago |
0-30 30 seconds |
28187 |
vihdzp author:vihdzp |
feat: archimedean classes of rationals |
We prove some lemmas relating `ArchimedeanClass` to `ℚ` and other archimedean fields.
---
- [x] depends on: #28179
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
64/5 |
Mathlib/Algebra/Order/Archimedean/Class.lean,Mathlib/Algebra/Order/Ring/Archimedean.lean,Mathlib/Order/Antisymmetrization.lean |
3 |
8 |
['github-actions', 'kckennylau', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'vihdzp', 'wwylele'] |
riccardobrasca assignee:riccardobrasca |
0-77846 21 hours ago |
11-25375 11 days ago |
11-29872 11 days |
28802 |
grunweg author:grunweg |
feat: a tactic linter for continuity/measurability which can be `fun_prop` |
---
Let's see if this finds further locations in mathlib :tada:
This PR also runs the linter in mathlib by default. I strongly think this is a good idea --- but leaves all kinds of fun questions around "where do you import this linter best". Opinions on this welcome; this PR is a first start (but no more).
[](https://gitpod.io/from-referrer/)
|
large-import
awaiting-CI
t-meta
|
144/26 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Basic.lean,Mathlib/Tactic/TacticAnalysis/Declarations.lean,Mathlib/Tactic/TacticAnalysis/FunProp.lean,MathlibTest/TacticAnalysis2.lean |
6 |
11 |
['Vierkantor', 'github-actions', 'grunweg', 'mathlib4-merge-conflict-bot'] |
nobody |
0-76256 21 hours ago |
2-64602 2 days ago |
0-260 4 minutes |
29177 |
scholzhannah author:scholzhannah |
feat: a subcomplex of a classical CW complex is a CW complex |
This PR proves that any subcomplex of a (relative classical) CW complex is again a CW complex.
---
While the definition of subcomplexes is in a different file (`Toplogy.CWComplex.Classical.Basic`) we create a separate file for subcomplexes because we will later add more proofs (such as the type of subcomplexes of a CW complex being a `CompletelyDistribLattice`).
[](https://gitpod.io/from-referrer/)
|
t-topology
delegated
|
204/8 |
Mathlib.lean,Mathlib/Topology/CWComplex/Classical/Basic.lean,Mathlib/Topology/CWComplex/Classical/Subcomplex.lean,docs/references.bib |
4 |
23 |
['ADedecker', 'github-actions', 'mathlib-bors', 'scholzhannah'] |
ocfnash assignee:ocfnash |
0-76208 21 hours ago |
0-76208 21 hours ago |
11-73 11 days |
29590 |
uniwuni author:uniwuni |
chore(Algebra/Group/Submonoid/Membership): fix outdated docs |
removes two declarations from the doc header that are no longer part of the file and quickly explains `Submonoid.powers` and `AddSubmonoid.multiples`
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
easy
label:t-algebra$ |
3/2 |
Mathlib/Algebra/Group/Submonoid/Membership.lean |
1 |
2 |
['github-actions', 'uniwuni'] |
nobody |
0-76139 21 hours ago |
0-76139 21 hours ago |
0-76188 21 hours |
29587 |
uniwuni author:uniwuni |
feat(GroupTheory/Finiteness): define finitely generated semigroups |
We define finitely generated semigroups and basics similarly to monoids and groups and prove that semigroups and monoids remain finitely generated when a congruence is quotiented out. This will be important when further developing semigroup theory.
---
[](https://gitpod.io/from-referrer/)
|
|
259/14 |
Mathlib/Algebra/Group/Submonoid/Defs.lean,Mathlib/GroupTheory/Finiteness.lean |
2 |
3 |
['github-actions', 'plp127', 'uniwuni'] |
nobody |
0-75776 21 hours ago |
0-81100 22 hours ago |
0-81081 22 hours |
29593 |
Vierkantor author:Vierkantor |
chore(*): replace `simp? says` with `simp only` |
Replace the output of `simp? says` with a `simp only` where the proof does not become less readable, and then golf the result by trying to drop lemmas from the simp set, or even replace it outright with (`simp_`)`rw`.
This is a weaker form of #29442.
---
[](https://gitpod.io/from-referrer/)
|
|
17/25 |
Mathlib/Algebra/Homology/Augment.lean,Mathlib/Algebra/MvPolynomial/Rename.lean,Mathlib/Algebra/Polynomial/Coeff.lean,Mathlib/Computability/PartrecCode.lean,Mathlib/Computability/TMToPartrec.lean,Mathlib/Data/List/Sigma.lean,Mathlib/Data/Ordmap/Ordset.lean,Mathlib/Data/PFunctor/Multivariate/M.lean,Mathlib/Data/QPF/Multivariate/Constructions/Fix.lean,Mathlib/Data/Seq/Parallel.lean,Mathlib/Data/Set/Enumerate.lean,Mathlib/Data/WSeq/Productive.lean,Mathlib/Data/WSeq/Relation.lean,Mathlib/GroupTheory/CoprodI.lean,Mathlib/MeasureTheory/Integral/Lebesgue/Add.lean,Mathlib/NumberTheory/Zsqrtd/Basic.lean |
16 |
1 |
['github-actions'] |
nobody |
0-74223 20 hours ago |
0-74293 20 hours ago |
0-74274 20 hours |
29578 |
vlad902 author:vlad902 |
feat(SimpleGraph): remove finiteness assumption from `isEmpty_of_chromaticNumber_eq_zero` |
|
t-combinatorics
easy
awaiting-author
|
11/11 |
Mathlib/Combinatorics/SimpleGraph/Coloring.lean |
1 |
5 |
['github-actions', 'grunweg', 'themathqueen', 'vlad902'] |
nobody |
0-73923 20 hours ago |
1-7066 1 day ago |
0-9935 2 hours |
29401 |
eric-wieser author:eric-wieser |
feat: more lemmas about `Matrix.vecMulVec` |
The most interesting of these is `(vecMulVec u v).det = 0`.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
54/0 |
Mathlib/Data/Matrix/Mul.lean,Mathlib/LinearAlgebra/Matrix/Determinant/Basic.lean,Mathlib/LinearAlgebra/Matrix/RowCol.lean,Mathlib/LinearAlgebra/Matrix/Trace.lean |
4 |
1 |
['github-actions', 'llllvvuu'] |
nobody |
0-73602 20 hours ago |
1-44094 1 day ago |
5-78394 5 days |
28693 |
faenuccio author:faenuccio |
feat(Analysis.Normed.Module.Milman-Pettis): add Milman-Pettis theorem |
We add the Milman-Pettis theorem stating that an uniformly convex Banach space is reflexive.
---
[](https://gitpod.io/from-referrer/)
|
t-analysis
WIP
|
279/0 |
Mathlib/Analysis/Convex/Uniform.lean,Mathlib/Analysis/Normed/Module/Dual.lean,Mathlib/Analysis/Normed/Module/Milman-Pettis.lean,Mathlib/Topology/Algebra/Module/WeakDual.lean |
4 |
3 |
['faenuccio', 'github-actions', 'grunweg'] |
nobody |
0-72009 20 hours ago |
23-76633 23 days ago |
0-1 1 second |
29594 |
faenuccio author:faenuccio |
feat(Algebra.Order.GroupWithZero.WithZero): add multiplicativity |
Branched out of #26588
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
6/2 |
Mathlib/Algebra/Order/GroupWithZero/WithZero.lean |
1 |
4 |
['YaelDillies', 'faenuccio', 'github-actions', 'pechersky'] |
nobody |
0-71741 19 hours ago |
0-72507 20 hours ago |
0-72545 20 hours |
29087 |
dupuisf author:dupuisf |
feat: Define strictly positive operators (i.e. positive definite) |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
203/21 |
Mathlib.lean,Mathlib/Algebra/Algebra/StrictPositivity.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Order.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Unital.lean,Mathlib/Analysis/SpecialFunctions/ContinuousFunctionalCalculus/ExpLog.lean,Mathlib/Analysis/SpecialFunctions/ContinuousFunctionalCalculus/Rpow/Basic.lean,Mathlib/Topology/UniformSpace/Real.lean |
7 |
10 |
['dupuisf', 'github-actions', 'themathqueen'] |
kim-em assignee:kim-em |
0-71629 19 hours ago |
13-43232 13 days ago |
13-43214 13 days |
28958 |
faenuccio author:faenuccio |
feat: add Nontrivial instance for linear maps |
Show that the space of `K`-linear maps between two non-trivial `K`-vector spaces is nontrivial, and that the space of continuous linear maps between two non-trivial normed spaces over an RCLike field `k` is nontrivial. The requirement that `k` be RCLike is needed because this is the setting in which Hahn-Banach is currently proven.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-analysis
awaiting-author
label:t-algebra$ |
28/9 |
Mathlib/Analysis/Normed/Module/Span.lean,Mathlib/Analysis/NormedSpace/HahnBanach/Extension.lean,Mathlib/LinearAlgebra/Basis/VectorSpace.lean,Mathlib/MeasureTheory/Function/AEEqOfIntegral.lean |
4 |
12 |
['ADedecker', 'faenuccio', 'github-actions', 'mathlib4-merge-conflict-bot', 'plp127'] |
nobody |
0-70724 19 hours ago |
0-70996 19 hours ago |
8-814 8 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 |
19/0 |
Mathlib/Topology/LocallyFinsupp.lean |
1 |
14 |
['Raph-DG', 'github-actions', 'jcommelin', 'kckennylau'] |
jcommelin assignee:jcommelin |
0-70357 19 hours ago |
4-75964 4 days ago |
76-54897 76 days |
27964 |
smmercuri author:smmercuri |
refactor(AbsoluteValue): generalise equivalence to non-real valued absolute values |
- Abstract the definition of `AbsoluteValue.IsEquiv` to any `AbsoluteValue R S` via preservation of partial orders (previously defined only for real absolute value using the power relation `(v .)^c = w`)
- Show `AbsoluteValue.IsEquiv` is equivalent to the power definition when the values are real
- Two inequivalent absolute values `v` and `w` have a point `x` at which `1 < v x` and `w x < 1`
---
This PR continues the work from #22100.
Original PR: https://github.com/leanprover-community/mathlib4/pull/22100 |
maintainer-merge
t-algebra
t-analysis
label:t-algebra$ |
212/44 |
Mathlib/Algebra/Order/AbsoluteValue/Basic.lean,Mathlib/Analysis/AbsoluteValue/Equivalence.lean,Mathlib/NumberTheory/Ostrowski.lean |
3 |
63 |
['MichaelStollBayreuth', 'YaelDillies', 'github-actions', 'smmercuri'] |
YaelDillies assignee:YaelDillies |
0-70015 19 hours ago |
0-75290 20 hours ago |
31-20025 31 days |
29598 |
xroblot author:xroblot |
feat(NumberField): two ring-isomorphic number fields have the same discriminant |
---
[](https://gitpod.io/from-referrer/)
|
t-number-theory
easy
|
4/0 |
Mathlib/NumberTheory/NumberField/Discriminant/Defs.lean |
1 |
1 |
['github-actions'] |
nobody |
0-68114 18 hours ago |
0-68299 18 hours ago |
0-68293 18 hours |
29597 |
alreadydone author:alreadydone |
feat(Algebra): preliminaries for ring structure on `AddLocalization` |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
77/5 |
Mathlib/Algebra/Module/End.lean,Mathlib/Algebra/Order/Nonneg/Basic.lean,Mathlib/Algebra/Order/Nonneg/Ring.lean,Mathlib/Algebra/Ring/Invertible.lean,Mathlib/LinearAlgebra/TensorProduct/Basic.lean |
5 |
1 |
['github-actions'] |
nobody |
0-67086 18 hours ago |
0-67086 18 hours ago |
0-67068 18 hours |
26357 |
javra author:javra |
feat(CategoryTheory): linear categories as `ModuleCat R`-enriched categories |
Continues #23826.
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-category-theory
|
197/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 |
9 |
['adamtopaz', 'github-actions', 'javra'] |
adamtopaz assignee:adamtopaz |
0-66901 18 hours ago |
11-67785 11 days ago |
75-952 75 days |
28493 |
gasparattila author:gasparattila |
feat: topological affine spaces |
This PR adds a typeclass `IsTopologicalAddTorsor` for topological affine spaces and generalizes several results which currently assume `NormedAddTorsor`.
---
[](https://gitpod.io/from-referrer/)
|
large-import
new-contributor
t-analysis
t-topology
|
403/310 |
Mathlib/Algebra/AddTorsor/Basic.lean,Mathlib/Analysis/Calculus/AddTorsor/AffineMap.lean,Mathlib/Analysis/Complex/AbsMax.lean,Mathlib/Analysis/Normed/Affine/AddTorsor.lean,Mathlib/Analysis/Normed/Affine/ContinuousAffineMap.lean,Mathlib/Analysis/Normed/Affine/Convex.lean,Mathlib/Analysis/Normed/Affine/Isometry.lean,Mathlib/Analysis/Normed/Group/AddTorsor.lean,Mathlib/Analysis/Normed/Module/FiniteDimension.lean,Mathlib/Analysis/Normed/Operator/Banach.lean,Mathlib/Analysis/RCLike/Lemmas.lean,Mathlib/Geometry/Euclidean/Projection.lean,Mathlib/Geometry/Euclidean/Triangle.lean,Mathlib/Topology/Algebra/Affine.lean,Mathlib/Topology/Algebra/ContinuousAffineMap.lean,Mathlib/Topology/Algebra/Group/Pointwise.lean |
16 |
6 |
['ADedecker', 'github-actions', 'mathlib4-merge-conflict-bot'] |
ADedecker assignee:ADedecker |
0-66335 18 hours ago |
8-64341 8 days ago |
26-74638 26 days |
29592 |
themathqueen author:themathqueen |
feat(Analysis/SpecialFunctions/CFC/Rpow): `0 ≤ a` iff `a = star b * b` for some `b` |
It can sometimes be convenient to directly have this form for non-negative elements.
---
[](https://gitpod.io/from-referrer/)
|
t-analysis |
4/0 |
Mathlib/Analysis/SpecialFunctions/ContinuousFunctionalCalculus/Rpow/Basic.lean |
1 |
2 |
['github-actions', 'j-loreaux'] |
nobody |
0-66217 18 hours ago |
0-74239 20 hours ago |
0-74284 20 hours |
29144 |
ADedecker author:ADedecker |
feat: some lemmas about closed maps |
This is a compilation of (1) some observations by @PatrickMassot and (2) some lemmas written by @AntoineChambert-Loir and I for a specific application, which turned out to have a nice proof using (1). The most interesting results are:
- `isClosedMap_iff_kernImage`: a map is closed iff the [Set.kernImage](https://leanprover-community.github.io/mathlib4_docs/Mathlib/Data/Set/Operations.html#Set.kernImage) of any ***open set*** is open (+ similar result for open maps)
- `isClosedMap_iff_comap_nhds_le`: as a consequence, the map `f` is closed iff for any `y`, one has `comap f (𝓝 y) ≤ 𝓝ˢ (f ⁻¹' {y})` (with equality if `f` is also continuous)
- `IsClosedMap.eventually_nhds_fiber` is a restatement of this in `eventually` terms: assuming `f` is closed, if some property holds in the neighborhood of the fiber at `y₀`, then it holds on the fiber at `y` for all `y` close enough to `y₀`.
---
I expect importing issues, but let's see...
[](https://gitpod.io/from-referrer/)
|
t-topology
delegated
|
99/2 |
Mathlib/Topology/Maps/Basic.lean |
1 |
6 |
['github-actions', 'j-loreaux', 'mathlib-bors'] |
j-loreaux assignee:j-loreaux |
0-65664 18 hours ago |
3-51141 3 days ago |
10-22183 10 days |
29599 |
fmortimore author:fmortimore |
feat(Order): bourbaki-witt theorem |
This adds a new file with a proof of the Bourbaki-Witt Theorem
Motivation: formalising one of Wiedijk's 1000+ theorems
---
[](https://gitpod.io/from-referrer/)
|
new-contributor |
4/0 |
Mathlib.lean,docs/1000.yaml |
2 |
1 |
['github-actions'] |
nobody |
0-65479 18 hours ago |
0-65537 18 hours ago |
0-65527 18 hours |
29600 |
xroblot author:xroblot |
feat(IsPrimitiveRoot): add `adjoin_pair_eq` |
The sub-algebra generated by two roots of unity of order `k₁` and `k₂` resp. is the same as the one
generated by a single root of unity of order `lcm k₁ k₂`.
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory |
30/0 |
Mathlib/RingTheory/RootsOfUnity/PrimitiveRoots.lean |
1 |
1 |
['github-actions'] |
nobody |
0-64888 18 hours ago |
0-64899 18 hours ago |
0-64937 18 hours |
27429 |
smorel394 author:smorel394 |
feat(RepresentationTheory/FinGroupCharZero): applications of Maschke's theorem |
Prove some properties of representations that follow from Maschke's theorem:
* If `G` is a finite group whose order is invertible in a field `k`, then every object of `Rep k G` (resp. `FDRep k G`) is injective and projective.
* For an object `V` of `FDRep k G`, when `k` is an algebraically closed field in which the order of `G` is invertible:
(1) `V` is simple if and only `V ⟶ V` is a `k`-vector space of dimension `1` (`FDRep.simple_iff_end_is_rank_one`);
(2) When `k` is characteristic zero, `V` is simple if and only if `∑ g : G, V.character g * V.character g⁻¹ = Fintype.card G` (`FDRep.simple_iff_char_is_norm_one`).
Note: This used to be #27165, but it was closed for some reason I don't understand.
- [x] depends on: #27154
- [x] depends on: #27134
- [x] depends on: #27125
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
169/0 |
Mathlib.lean,Mathlib/Algebra/Category/FGModuleCat/Abelian.lean,Mathlib/RepresentationTheory/FinGroupCharZero.lean |
3 |
4 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
0-64645 17 hours ago |
0-67059 18 hours ago |
0-67414 18 hours |
29319 |
Louddy author:Louddy |
feat(SkewMonoidAlgebra): Modifying elements of skew monoid algebra at exactly one point (erase and update) |
Basic results on updating/erasing an element of a skew monoid algebras using one point of the domain. Similar to `Finsupp.erase` and `Finsupp.update`
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
awaiting-author
label:t-algebra$ |
146/0 |
Mathlib.lean,Mathlib/Algebra/SkewMonoidAlgebra/Single.lean |
2 |
4 |
['github-actions', 'ocfnash'] |
ocfnash assignee:ocfnash |
0-64633 17 hours ago |
0-64633 17 hours ago |
9-7446 9 days |
29501 |
Vierkantor author:Vierkantor |
test(TacticAnalysis): ensure `classical`'s effects are picked up |
This test case currently fails, and needs a fix to the `classical` tactic in the standard library:
- [ ] depends on: https://github.com/leanprover/lean4/pull/10332
---
[](https://gitpod.io/from-referrer/)
|
blocked-by-core-PR |
10/0 |
MathlibTest/TacticAnalysis.lean |
1 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
0-64504 17 hours ago |
0-64507 17 hours ago |
0-0 0 seconds |
29182 |
euprunin author:euprunin |
chore: remove redundant `congr` invocations |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
3/15 |
Mathlib/Algebra/BigOperators/Finprod.lean,Mathlib/Algebra/Homology/HomotopyCategory/HomComplexShift.lean,Mathlib/Algebra/Module/LocalizedModule/Basic.lean,Mathlib/Algebra/MvPolynomial/Basic.lean,Mathlib/Algebra/Polynomial/Coeff.lean,Mathlib/Algebra/Polynomial/Roots.lean,Mathlib/Algebra/Polynomial/Splits.lean |
7 |
23 |
['euprunin', 'github-actions', 'grunweg', 'leanprover-bot', 'leanprover-community-mathlib4-bot'] |
nobody |
0-63548 17 hours ago |
0-63548 17 hours ago |
8-58744 8 days |
28100 |
themathqueen author:themathqueen |
feat(LinearAlgebra/Matrix): algebra automorphisms on matrices are inner |
Characterization of automorphisms on matrices: for any algebra automorphism `f : Matrix n n R ≃ₐ[R] Matrix n n R`, there exists an invertible matrix `T` such that `f a = T * a * T⁻¹` for all `a`.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
awaiting-author
label:t-algebra$ |
74/0 |
Mathlib/LinearAlgebra/Matrix/GeneralLinearGroup/Basic.lean |
1 |
27 |
['Whysoserioushah', 'eric-wieser', 'github-actions', 'mathlib4-merge-conflict-bot', 'themathqueen'] |
Vierkantor assignee:Vierkantor |
0-62440 17 hours ago |
0-62464 17 hours ago |
34-16869 34 days |
29601 |
jt496 author:jt496 |
feat(SimpleGraph/Walk): add missing results involving `getVert` / `takeUntil` |
Add some missing lemmas involving `getVert` / `takeUntil`.
In particular `getVert_le_length_takeUntil_eq_iff` which says that if `p` is a walk containing the vertex `u` then `n = (p.takeUntil u h).length` is the smallest `n` such that `p.getVert n = u`.
---
[](https://gitpod.io/from-referrer/)
|
t-combinatorics |
47/61 |
Mathlib/Combinatorics/SimpleGraph/Connectivity/WalkDecomp.lean,Mathlib/Combinatorics/SimpleGraph/Walk.lean |
2 |
1 |
['github-actions'] |
nobody |
0-61474 17 hours ago |
0-61537 17 hours ago |
0-61550 17 hours |
29436 |
eric-wieser author:eric-wieser |
feat: a better version of `LinearOrder.lift` |
This adds the following, which do not construct any new data and instead assume compatibility:
* `Function.Injective.preorder` (a generalization of `PreOrder.lift`)
* `Function.Injective.partialOrder` (a generalization of `PartialOrder.lift`)
* `Function.Injective.linearOrder` (a generalization of `LinearOrder.liftWithOrd` and the other three variants)
The following existing constructions are modified to do the same (and confusingly no longer assume injectivity):
* `Function.Injective.isOrderedAddMonoid`
* `Function.Injective.isOrderedRing`
* `Function.Injective.isStrictOrderedRing`
This fixes the instance diamond in [#mathlib4 > Instance diamond in DecidableEq Fin @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Instance.20diamond.20in.20DecidableEq.20Fin/near/538119386) (which was discovered in #29418), by reusing the existing `Decidable` instance rather than constructing defeq-but-only-without-smart-unfolding instance from scratch.
---
[](https://gitpod.io/from-referrer/)
|
maintainer-merge
t-order
|
200/173 |
Counterexamples/MapFloor.lean,Mathlib/Algebra/Group/Subgroup/Order.lean,Mathlib/Algebra/Module/Submodule/Order.lean,Mathlib/Algebra/Order/Field/Subfield.lean,Mathlib/Algebra/Order/GroupWithZero/Canonical.lean,Mathlib/Algebra/Order/Monoid/Basic.lean,Mathlib/Algebra/Order/Monoid/Submonoid.lean,Mathlib/Algebra/Order/Monoid/Units.lean,Mathlib/Algebra/Order/Nonneg/Ring.lean,Mathlib/Algebra/Order/Ring/InjSurj.lean,Mathlib/Algebra/Ring/Subring/Order.lean,Mathlib/Algebra/Ring/Subsemiring/Order.lean,Mathlib/Analysis/Seminorm.lean,Mathlib/Order/Basic.lean,Mathlib/Order/Fin/Basic.lean,Mathlib/Order/Lattice.lean |
16 |
15 |
['YaelDillies', 'eric-wieser', 'github-actions', 'plp127'] |
nobody |
0-61243 17 hours ago |
0-61262 17 hours ago |
1-43232 1 day |
29391 |
eric-wieser author:eric-wieser |
feat: more connections between `TensorProduct` and `map₂` |
The new lemmas about `map₂` are analogous to the lemmas about `Set.image2`.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
50/10 |
Mathlib/Algebra/Lie/TensorProduct.lean,Mathlib/Algebra/Module/Submodule/Bilinear.lean,Mathlib/LinearAlgebra/TensorProduct/Basic.lean,Mathlib/LinearAlgebra/TensorProduct/Quotient.lean |
4 |
1 |
['github-actions'] |
nobody |
0-61130 16 hours ago |
6-40304 6 days ago |
6-40286 6 days |
29602 |
CBirkbeck author:CBirkbeck |
Setup the Infinite conditional sums API |
This is an attempt to develop some conditional infinite sum API
---
[](https://gitpod.io/from-referrer/)
|
|
382/0 |
Mathlib/NumberTheory/IccSums.lean,Mathlib/Topology/Algebra/InfiniteConditionalSum/Basic.lean,Mathlib/Topology/Algebra/Monoid/Defs.lean |
3 |
1 |
['github-actions'] |
nobody |
0-60724 16 hours ago |
0-60982 16 hours ago |
0-0 0 seconds |
26345 |
mans0954 author:mans0954 |
feature(Analysis/LocallyConvex/Polar): Bipolar theorem |
The bipolar theorem states that the polar of the polar of a set `s` is equal to the closed absolutely convex hull of `s`.
The argument here follows Conway, Chapter V. 1.8.
This PR continues the work from #20843.
Original PR: https://github.com/leanprover-community/mathlib4/pull/20843
- [x] depends on: #27316 |
large-import
t-analysis
awaiting-author
|
201/27 |
Mathlib.lean,Mathlib/Analysis/LocallyConvex/AbsConvex.lean,Mathlib/Analysis/LocallyConvex/Bipolar.lean,Mathlib/Analysis/Normed/Module/Dual.lean,Mathlib/Topology/Algebra/Module/StrongTopology.lean,Mathlib/Topology/Algebra/Module/WeakBilin.lean |
6 |
n/a |
['JonBannon', 'eric-wieser', 'faenuccio', 'github-actions', 'j-loreaux', 'leanprover-community-bot-assistant', 'mans0954', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
0-59385 16 hours ago |
unknown |
unknown |
28115 |
bwangpj author:bwangpj |
feat(AlgebraicGeometry/EllipticCurve): reduction of elliptic curves |
Define the reduction of elliptic curves over the fraction field of a DVR, following Silverman.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-algebraic-geometry
|
251/0 |
Mathlib.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Reduction.lean,Mathlib/GroupTheory/ArchimedeanDensely.lean |
3 |
34 |
['Multramate', 'adamtopaz', 'bwangpj', 'github-actions', 'kbuzzard'] |
adamtopaz assignee:adamtopaz |
0-59205 16 hours ago |
2-45784 2 days ago |
35-39995 35 days |
27216 |
D-Thomine author:D-Thomine |
feat(Cardinal/Finite): ENat powers and cardinality |
This PR continues the work from #25574.
Original PR: https://github.com/leanprover-community/mathlib4/pull/25574 |
t-algebra label:t-algebra$ |
205/6 |
Mathlib.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/Data/ENat/Pow.lean,Mathlib/SetTheory/Cardinal/Finite.lean |
4 |
17 |
['D-Thomine', 'eric-wieser', 'github-actions', 'kbuzzard', 'mathlib4-merge-conflict-bot'] |
kbuzzard assignee:kbuzzard |
0-58818 16 hours ago |
23-63936 23 days ago |
52-71175 52 days |
28818 |
NotWearingPants author:NotWearingPants |
feat(Data/Setoid/Basic): add theorems about lifting a function to its kernel |
Currently `ker_lift_injective` and `quotientKerEquivOfRightInverse` lift `f` to `ker f` in their definition.
This PR makes this function available as `Setoid.ker_lift f` and adds a few more theorems about it.
---
[](https://gitpod.io/from-referrer/)
|
t-data
new-contributor
easy
|
28/13 |
Counterexamples/AharoniKorman.lean,Mathlib/Data/Setoid/Basic.lean |
2 |
3 |
['NotWearingPants', 'github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
0-58359 16 hours ago |
0-58411 16 hours ago |
18-73355 18 days |
29241 |
yoh-tanimoto author:yoh-tanimoto |
feat(Analysis/InnerProductSpace/Orthogonal): add duplicates for `ClosedSubmodule` |
add duplicates of definitions and API's for `ClosedSubmodule` in an `InnerProductSpace`.
motivation: when one considers a Hilbert space (`CompleteSpace`), it is more natural to consider `ClosedSubmodule`s. They form a complete lattice and satisfy `sup_orthogonal` #29243.
- [x] depends on: #29230 for `Lattice` `CompleteLattice` |
|
191/0 |
Mathlib/Analysis/InnerProductSpace/Orthogonal.lean |
1 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
0-58092 16 hours ago |
0-64467 17 hours ago |
0-64953 18 hours |
29235 |
yoh-tanimoto author:yoh-tanimoto |
feat(Topology/Algebra/Module/ClosedSubmodule): add `mapEquiv`, a variation of `ClosedSubmodule.map` for CLE |
add `ClosedSubmodule.map` for continuous linear equivalence. In this case, a closed map is mapped to a closed map, so the definitions are easier and behave nicely with `closure` and `⊔`.
motivation: needed to define standard subspaces in a Hilbert space (scalar multiplication by `Complex.I`) #29251
https://ems.press/content/serial-article-files/48171
- [x] depends on: #29230 for `Lattice` `CompleteLattice` |
t-topology |
69/1 |
Mathlib/Topology/Algebra/Module/ClosedSubmodule.lean |
1 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
0-58080 16 hours ago |
0-64465 17 hours ago |
0-66756 18 hours |
27043 |
wwylele author:wwylele |
feat(Algebra/Order): Hahn embedding theorem, part 1 |
Part 1 of Hahn embedding theorem, or the core part of it. This proves that one can embed an ordered module in HahnSeries.
To obtain the full Hahn embedding theorem, one needs to specialize the coefficient of HahnSeries to Real as a module over Rat, and compose with another embedding from ordered group to ordered module. These will be in part 2
There is a debatable design here: throughout the file, all lemmas uses an input `HahnEmbedding.Seed`. Because the the final theorem is an existence theorem without specifying what `HahnEmbedding.Seed` is used, it is possible to `Classical.choose` a seed from the very beginning (provided `R = Real` ), and the entire file will just use the same chosen seed. Overall, choosing everything from the beginning will likely make the code a little bit more concise.
I decided against choosing anything till the final step, for the reason that such choice is not canonical for an arbitrary module, and there may be future use of this construction with more canonical choice for specific modules. Examples are:
- if the input is a `HahnSeries Γ R`, the canonical choice for the `stratum` would be `HahnSeries.single`
- for the field version of Hahn embedding theorem ("every linearly ordered field can be embedded in `HahnSeries` as a field", not implemented), the canonical choice should ensure that all `stratum` form a graded ring, and the `coeff` should map `(1 : M)` to `(1 : R)`.
But if the argument is not strong enough, I am OK with converting everything to a classical choose.
---
- [x] depends on: #25970
- [x] depends on: #27054
- [x] depends on: #27055
- [x] depends on: #27711
- [x] depends on: #27885
- [x] depends on: #28136
- [x] depends on: #28449
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
1016/0 |
Mathlib.lean,Mathlib/Algebra/Order/Module/HahnEmbedding.lean,docs/references.bib |
3 |
85 |
['YaelDillies', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'vihdzp', 'wwylele'] |
nobody |
0-55942 15 hours ago |
0-55943 15 hours ago |
10-39895 10 days |
27270 |
EtienneC30 author:EtienneC30 |
chore: turn WithLp into a structure |
Turn `WithLp` into a one field structure, as was suggested many times on Zulip and discussed here: https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/defeq.20abuse.20in.20.60WithLp.60/near/526234806.
Here is what this PR does:
- The instances on `WithLp p α` which were defeq to those on `α` (algebraic instances, topology, uniformity, bornology) are now pulled back from `α` along `WithLp.equiv p α`. A few declarations are added to ease the process, such as versions of `WithLp.equiv` as a homeomorphism or a uniform isomorphism.
- It introduces some definitions to equip `α × β` with the Lp distance, and similarly for `Π i, α i`. This is then used to define relevant instances on type synonyms, such as for matrix norms.
- The PR fixes all the defeq abuses (which break obviously).
---
- [x] depends on: #28469
- [x] depends on: #28470
- [x] depends on: #28471
[](https://gitpod.io/from-referrer/)
|
large-import
t-analysis
|
619/407 |
Archive/Hairer.lean,Mathlib/Algebra/Module/ZLattice/Covolume.lean,Mathlib/Analysis/CStarAlgebra/Matrix.lean,Mathlib/Analysis/Calculus/FDeriv/WithLp.lean,Mathlib/Analysis/InnerProductSpace/PiL2.lean,Mathlib/Analysis/InnerProductSpace/Positive.lean,Mathlib/Analysis/InnerProductSpace/ProdL2.lean,Mathlib/Analysis/InnerProductSpace/Spectrum.lean,Mathlib/Analysis/Matrix.lean,Mathlib/Analysis/Normed/Algebra/TrivSqZeroExt.lean,Mathlib/Analysis/Normed/Algebra/UnitizationL1.lean,Mathlib/Analysis/Normed/Lp/LpEquiv.lean,Mathlib/Analysis/Normed/Lp/MeasurableSpace.lean,Mathlib/Analysis/Normed/Lp/PiLp.lean,Mathlib/Analysis/Normed/Lp/ProdLp.lean,Mathlib/Analysis/Normed/Lp/WithLp.lean,Mathlib/Analysis/Quaternion.lean,Mathlib/Analysis/RCLike/Inner.lean,Mathlib/Analysis/SpecialFunctions/Gaussian/FourierTransform.lean,Mathlib/Combinatorics/Additive/AP/Three/Behrend.lean,Mathlib/Geometry/Euclidean/Angle/Unoriented/CrossProduct.lean,Mathlib/Geometry/Manifold/Instances/Icc.lean,Mathlib/Geometry/Manifold/Instances/Real.lean,Mathlib/LinearAlgebra/Matrix/Hermitian.lean,Mathlib/LinearAlgebra/Matrix/PosDef.lean,Mathlib/LinearAlgebra/Matrix/Spectrum.lean,Mathlib/MeasureTheory/Measure/Haar/InnerProductSpace.lean,Mathlib/MeasureTheory/Measure/Haar/OfBasis.lean,Mathlib/MeasureTheory/Measure/Lebesgue/VolumeOfBalls.lean,Mathlib/MeasureTheory/SpecificCodomains/WithLp.lean,Mathlib/NumberTheory/NumberField/CanonicalEmbedding/Basic.lean,Mathlib/NumberTheory/NumberField/Ideal/Asymptotics.lean |
32 |
45 |
['EtienneC30', 'eric-wieser', 'github-actions', 'j-loreaux', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
j-loreaux assignee:j-loreaux |
0-55573 15 hours ago |
0-57507 15 hours ago |
29-6139 29 days |
25831 |
ScottCarnahan author:ScottCarnahan |
feat (RingTheory/HahnSeries): Powers of a binomial |
This PR introduces powers of a binomial `single g 1 - single g' 1` in a Hahn series, where the powers take values in a binomial ring. These series behave as one would expect with respect to addition of powers, and comparison with natural number powers. They are often used in the theory of vertex algebras.
---
- [x] depends on: #25830
- [x] depends on: #27497
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #24102.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/24102* |
t-ring-theory |
111/0 |
Mathlib.lean,Mathlib/RingTheory/HahnSeries/Binomial.lean,Mathlib/RingTheory/HahnSeries/HEval.lean,Mathlib/RingTheory/HahnSeries/Multiplication.lean |
4 |
8 |
['github-actions', 'kbuzzard', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
kbuzzard assignee:kbuzzard |
0-54089 15 hours ago |
29-44366 29 days ago |
29-45826 29 days |
27257 |
JovanGerb author:JovanGerb |
feat(LinearAlgebra/AffineSpace/Ordered): add `lineMap_le_lineMap_iff_of_lt'` |
I only need `lineMap_le_lineMap_iff_of_lt'`. The other lemmas are added for completeness.
---
[](https://gitpod.io/from-referrer/)
|
maintainer-merge
t-algebra
label:t-algebra$ |
44/0 |
Mathlib/LinearAlgebra/AffineSpace/Ordered.lean |
1 |
6 |
['JovanGerb', 'Ruben-VandeVelde', 'eric-wieser', 'github-actions', 'kbuzzard'] |
kbuzzard assignee:kbuzzard |
0-52664 14 hours ago |
12-1708 12 days ago |
26-19468 26 days |
26035 |
fbarroero author:fbarroero |
feat(Analysis/Polynomial/MahlerMeasure): the Mahler measure of a complex polynomial |
We introduce the Mahler measure of a complex polynomial and prove some basic facts.
---
[](https://gitpod.io/from-referrer/)
|
t-analysis |
127/1 |
Mathlib.lean,Mathlib/Analysis/Polynomial/MahlerMeasure.lean,Mathlib/MeasureTheory/Integral/CircleIntegral.lean |
3 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
sgouezel assignee:sgouezel |
0-52317 14 hours ago |
0-52335 14 hours ago |
86-53702 86 days |
26783 |
matthewjasper author:matthewjasper |
feat(RingTheory/Flat): Add theorems relating Submodule.torsion and Module.Flat |
Co-authored-by: Kevin Buzzard
---
This PR continues the work from #25334.
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
FLT
maintainer-merge
new-contributor
|
206/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 |
6 |
['github-actions', 'kbuzzard'] |
kbuzzard assignee:kbuzzard |
0-51937 14 hours ago |
0-51937 14 hours ago |
57-72863 57 days |
29582 |
YaelDillies author:YaelDillies |
chore: rename `_root_.prop` to `finite_prop` |
This was a surprising name!
---
[](https://gitpod.io/from-referrer/)
|
t-data |
1/1 |
Mathlib/Data/Fintype/EquivFin.lean |
1 |
9 |
['YaelDillies', 'eric-wieser', 'github-actions', 'grunweg', 'plp127'] |
nobody |
0-50924 14 hours ago |
0-75549 20 hours ago |
0-76882 21 hours |
29517 |
pechersky author:pechersky |
feat(RingTheory/Torsion): torsion = union of roots of unity |
with additional API for Associates and rootsOfUnity sups
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
136/19 |
Mathlib.lean,Mathlib/Algebra/GCDMonoid/Basic.lean,Mathlib/Algebra/Group/Subgroup/Lattice.lean,Mathlib/GroupTheory/OrderOfElement.lean,Mathlib/RingTheory/RootsOfUnity/Basic.lean,Mathlib/RingTheory/Torsion.lean |
6 |
4 |
['github-actions', 'kckennylau', 'pechersky'] |
nobody |
0-50650 14 hours ago |
2-47034 2 days ago |
2-47126 2 days |
29428 |
llllvvuu author:llllvvuu |
feat: generalize `LinearMap.finrank_maxGenEigenspace` |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
35/2 |
Mathlib/Algebra/Lie/Rank.lean,Mathlib/LinearAlgebra/Charpoly/Basic.lean,Mathlib/LinearAlgebra/Eigenspace/Basic.lean,Mathlib/LinearAlgebra/Eigenspace/Zero.lean,Mathlib/LinearAlgebra/Matrix/Charpoly/Basic.lean |
5 |
1 |
['github-actions'] |
nobody |
0-50109 13 hours ago |
5-19362 5 days ago |
5-19404 5 days |
29583 |
Ruben-VandeVelde author:Ruben-VandeVelde |
chore: tidy various files |
---
[](https://gitpod.io/from-referrer/)
|
maintainer-merge |
82/118 |
Counterexamples/CanonicallyOrderedCommSemiringTwoMul.lean,Mathlib/Algebra/GroupWithZero/Action/Hom.lean,Mathlib/Algebra/GroupWithZero/Range.lean,Mathlib/Algebra/Module/Submodule/Pointwise.lean,Mathlib/Algebra/Order/Module/Archimedean.lean,Mathlib/Algebra/QuadraticAlgebra.lean,Mathlib/Analysis/InnerProductSpace/Adjoint.lean,Mathlib/Analysis/InnerProductSpace/Positive.lean,Mathlib/CategoryTheory/Limits/Shapes/Multiequalizer.lean,Mathlib/CategoryTheory/Sites/SheafOfTypes.lean,Mathlib/Data/List/Indexes.lean,Mathlib/Data/List/Lemmas.lean,Mathlib/Data/List/OfFn.lean,Mathlib/Data/List/Pi.lean,Mathlib/Data/Nat/Bits.lean,Mathlib/Data/Nat/Factorial/NatCast.lean,Mathlib/LinearAlgebra/BilinearMap.lean,Mathlib/LinearAlgebra/Matrix/Spectrum.lean,Mathlib/NumberTheory/MulChar/Basic.lean,Mathlib/Probability/Moments/Variance.lean,Mathlib/RepresentationTheory/Basic.lean,Mathlib/RingTheory/Adjoin/Basic.lean,Mathlib/RingTheory/DedekindDomain/Ideal/Basic.lean,Mathlib/RingTheory/DividedPowers/RatAlgebra.lean,Mathlib/RingTheory/HahnSeries/Summable.lean,Mathlib/RingTheory/Ideal/Basic.lean,Mathlib/RingTheory/IntegralDomain.lean,Mathlib/RingTheory/LocalRing/Module.lean,Mathlib/RingTheory/Polynomial/Basic.lean,Mathlib/RingTheory/Polynomial/Content.lean,Mathlib/RingTheory/Polynomial/Cyclotomic/Basic.lean,Mathlib/Topology/Order/IsNormal.lean |
32 |
15 |
['Ruben-VandeVelde', 'github-actions', 'grunweg', 'uniwuni'] |
grunweg assignee:grunweg |
0-49478 13 hours ago |
0-49478 13 hours ago |
1-5705 1 day |
29513 |
grunweg author:grunweg |
fix(lint-style): parse linter options and load environment extensions correctly |
Parse options and load linter set extension correctly.
This fixes two issues:
- We never called the `toOptions` function that parses Lakefile options into a `Lean.Options` structure: the function we use instead is only meant for command-line options and doesn't handle the `weak.` prefix correctly.
- The way we load linter sets was incorrect: `withImportModules` doesn't update any environment extensions, and that is exactly what we use to store linter sets. We can replace it with `importModules` instead, but that is a bit less safe. It would be great if we had some sort of macro that can give us the environment at the point of elaboration instead.
TODO: that is now wrong, update the description to be correct!
---
- [x] depends on: #29584
- [x] depends on: #29585
- [x] depends on: #29586
[](https://gitpod.io/from-referrer/)
|
t-meta |
10/8 |
scripts/lint-style.lean |
1 |
7 |
['github-actions', 'grunweg', 'mathlib4-dependent-issues-bot'] |
nobody |
0-49179 13 hours ago |
0-49373 13 hours ago |
0-51973 14 hours |
26827 |
pechersky author:pechersky |
feat(Analysis/Normed/ValuativeRel): helper instance for NormedField |
---
[](https://gitpod.io/from-referrer/)
- [x] depends on: #26713
- [x] depends on: #26826
|
t-algebra
t-analysis
t-number-theory
label:t-algebra$ |
205/20 |
Mathlib.lean,Mathlib/Analysis/Normed/ValuativeRel.lean,Mathlib/Topology/Algebra/Valued/ValuativeRel.lean |
3 |
19 |
['ADedecker', 'adamtopaz', 'github-actions', 'kbuzzard', 'kckennylau', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'pechersky'] |
kbuzzard assignee:kbuzzard |
0-48717 13 hours ago |
30-67806 30 days ago |
67-47127 67 days |
27339 |
pechersky author:pechersky |
chore(RingTheory/Laurent): use WithZero.exp to golf statements and proofs about valuation on K((X)) |
Done as part of refactor of Valued in #27314. This PR does not change any definitions. Instead, uses `WithZero.exp` instead of coercion + Multiplicative.ofAdd. And some helper simp lemmas about valuations of RatFunc vis a vis LaurentSeries.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-number-theory
label:t-algebra$ |
73/75 |
Mathlib/FieldTheory/RatFunc/AsPolynomial.lean,Mathlib/RingTheory/LaurentSeries.lean |
2 |
7 |
['Louddy', 'faenuccio', 'github-actions', 'mathlib4-merge-conflict-bot', 'pechersky'] |
Vierkantor assignee:Vierkantor |
0-48645 13 hours ago |
14-59832 14 days ago |
49-5274 49 days |
29568 |
dagurtomas author:dagurtomas |
feat(CategoryTheory/Monoidal): more natural constructors for braided categories |
---
[](https://gitpod.io/from-referrer/)
|
t-category-theory |
282/0 |
Mathlib.lean,Mathlib/CategoryTheory/Functor/CurryingThree.lean,Mathlib/CategoryTheory/Monoidal/Braided/Multifunctor.lean |
3 |
3 |
['github-actions', 'joelriou'] |
nobody |
0-46396 12 hours ago |
1-20184 1 day ago |
1-20166 1 day |
29110 |
NotWearingPants author:NotWearingPants |
feat(Counterexamples): Euler's sum of powers conjecture |
feat(Counterexamples): Euler's sum of powers conjecture
---
[](https://gitpod.io/from-referrer/)
|
new-contributor |
159/0 |
Counterexamples.lean,Counterexamples/EulerSumOfPowers.lean |
2 |
34 |
['MichaelStollBayreuth', 'NotWearingPants', 'eric-wieser', 'github-actions', 'tb65536'] |
MichaelStollBayreuth assignee:MichaelStollBayreuth |
0-46254 12 hours ago |
0-49473 13 hours ago |
12-38267 12 days |
29512 |
grunweg author:grunweg |
feat: check for PR titles which do not start with "feat" etc. |
We ignore draft PRs and PRs with the WIP label.
The set of checks is intentionally kept small, and could be expanded in the
future.
---
More basic version of #16303: given that mathlib's statistics will use the PR kind, let's make sure PR kinds are somewhat appropriate.
[](https://gitpod.io/from-referrer/)
|
|
365/0 |
.github/build.in.yml,.github/workflows/bors.yml,.github/workflows/build.yml,.github/workflows/build_fork.yml,Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter/ValidatePRTitle.lean,lakefile.lean,scripts/README.md,scripts/check_title_labels.lean |
10 |
17 |
['bryangingechen', 'eric-wieser', 'github-actions', 'grunweg'] |
bryangingechen assignee:bryangingechen |
0-46216 12 hours ago |
2-65270 2 days ago |
2-65251 2 days |
28874 |
vasnesterov author:vasnesterov |
feat(Data/Seq): coinductive predicates for sequences |
* Prove `eq_of_bisim'` and `eq_of_bisim_strong` coinductive principles for equality.
* Develop API for a predicate `∀ x ∈ s, p x` where `s : Seq α`, including coinductive principle `all_coind`.
* Introduce the `Pairwise` predicate along with API and coinductive principles `Pairwise.coind` and `Pairwise.coind_trans`.
* Introduce `ENat`-valued length of a sequence, `length'`, along with minimal API.
* Move theorems about `length` from `Defs.lean` to `Basic.lean`.
* Prove a coinductive principle for a predicate `a.length' ≤ b.length'`.
All of these "coinductive principles" are stated in the form as similar as possible to inductive principles.
---
- [x] depends on: #26120
This PR is necessary for a new tactic (#28291), which computes the asymptotics of real functions.
[](https://gitpod.io/from-referrer/)
This PR continues the work from #20241.
Original PR: https://github.com/leanprover-community/mathlib4/pull/20241 |
large-import
t-data
|
420/48 |
Mathlib/Data/Seq/Basic.lean,Mathlib/Data/Seq/Defs.lean,Mathlib/Data/Stream/Init.lean |
3 |
25 |
['bryangingechen', 'eric-wieser', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'plp127', 'vasnesterov'] |
nobody |
0-42117 11 hours ago |
0-42278 11 hours ago |
14-70088 14 days |
29605 |
alreadydone author:alreadydone |
chore(Algebra): unbundle npow from Monoid |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
awaiting-CI
label:t-algebra$ |
436/300 |
Mathlib/Algebra/BigOperators/Group/List/Basic.lean,Mathlib/Algebra/BigOperators/Group/List/Defs.lean,Mathlib/Algebra/BigOperators/Group/Multiset/Defs.lean,Mathlib/Algebra/Divisibility/Basic.lean,Mathlib/Algebra/Group/Action/Defs.lean,Mathlib/Algebra/Group/Basic.lean,Mathlib/Algebra/Group/Commute/Basic.lean,Mathlib/Algebra/Group/Commute/Defs.lean,Mathlib/Algebra/Group/Defs.lean,Mathlib/Algebra/Group/Ext.lean,Mathlib/Algebra/Group/Fin/Basic.lean,Mathlib/Algebra/Group/Hom/Basic.lean,Mathlib/Algebra/Group/Hom/Defs.lean,Mathlib/Algebra/Group/InjSurj.lean,Mathlib/Algebra/Group/Int/Defs.lean,Mathlib/Algebra/Group/Nat/Defs.lean,Mathlib/Algebra/Group/Opposite.lean,Mathlib/Algebra/Group/PUnit.lean,Mathlib/Algebra/Group/Pi/Basic.lean,Mathlib/Algebra/Group/Semiconj/Basic.lean,Mathlib/Algebra/Group/Semiconj/Defs.lean,Mathlib/Algebra/Group/Submonoid/Defs.lean,Mathlib/Algebra/Group/Support.lean,Mathlib/Algebra/Group/Torsion.lean,Mathlib/Algebra/Group/TransferInstance.lean,Mathlib/Algebra/Group/TypeTags/Basic.lean,Mathlib/Algebra/Group/ULift.lean,Mathlib/Algebra/Group/Units/Defs.lean,Mathlib/Algebra/GroupWithZero/Action/Defs.lean,Mathlib/Algebra/GroupWithZero/Basic.lean,Mathlib/Algebra/GroupWithZero/Defs.lean,Mathlib/Algebra/GroupWithZero/Hom.lean,Mathlib/Algebra/GroupWithZero/Indicator.lean,Mathlib/Algebra/GroupWithZero/InjSurj.lean,Mathlib/Algebra/GroupWithZero/ULift.lean,Mathlib/Algebra/Order/Group/Multiset.lean,Mathlib/Algebra/Order/Group/Synonym.lean,Mathlib/Algebra/Order/Monoid/Basic.lean,Mathlib/Algebra/Order/Monoid/Unbundled/Pow.lean,Mathlib/Algebra/Order/Monoid/Unbundled/WithTop.lean,Mathlib/Algebra/Ring/Defs.lean,Mathlib/Algebra/Ring/GrindInstances.lean,Mathlib/Algebra/Ring/Torsion.lean,Mathlib/Data/DFinsupp/Defs.lean,Mathlib/Data/Int/Cast/Basic.lean,Mathlib/Data/Nat/Cast/Defs.lean,Mathlib/Data/Rat/Defs.lean |
47 |
1 |
['github-actions'] |
nobody |
0-41342 11 hours ago |
0-54290 15 hours ago |
0-2 2 seconds |
29411 |
llllvvuu author:llllvvuu |
feat(LinearAlgebra/Matrix/Rank): rank factorization |
The rank factorization derived from `Module.finBasis`.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
19/0 |
Mathlib/LinearAlgebra/Matrix/Rank.lean,Mathlib/LinearAlgebra/Matrix/ToLin.lean |
2 |
1 |
['github-actions'] |
nobody |
0-41301 11 hours ago |
5-47548 5 days ago |
5-47546 5 days |
27342 |
staroperator author:staroperator |
feat(ModelTheory): define linear and semilinear sets |
Separated from #27100. This PR defines the linear and semilinear sets for general `AddCommMonoid` and prove some basic properties.
---
- [x] depends on: #27099
- [x] depends on: #27085
- [x] depends on: #27341
---
[](https://gitpod.io/from-referrer/)
|
t-logic |
383/0 |
Mathlib.lean,Mathlib/ModelTheory/Arithmetic/Presburger/Semilinear/Defs.lean,docs/references.bib |
3 |
42 |
['JovanGerb', 'YaelDillies', 'awainverse', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'staroperator'] |
fpvandoorn assignee:fpvandoorn |
0-41142 11 hours ago |
0-67118 18 hours ago |
16-78947 16 days |
29607 |
wwylele author:wwylele |
feat(RingTheory): summability lemma for (Mv)PowerSeries |
About `PowerSeries.summable_of_tendsto_weightedOrder_atTop_nhds_top`, it surprised me that `PowerSeries.order` isn't implemented using `MvPowerSeries.order`, so I had to duplicate the proof for `MvPowerSeries` and `PowerSeries`. The other lemmas are also duplication instead of reusing the same proof, because it turned out piercing through defeq actually makes the code longer.
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory |
80/0 |
Mathlib/RingTheory/MvPowerSeries/PiTopology.lean,Mathlib/RingTheory/PowerSeries/PiTopology.lean |
2 |
1 |
['github-actions'] |
nobody |
0-40807 11 hours ago |
0-41082 11 hours ago |
0-41120 11 hours |
27053 |
tb65536 author:tb65536 |
(WIP) Galois group of `x^n - x - 1` |
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebra
WIP
label:t-algebra$ |
455/2 |
Mathlib/RingTheory/Polynomial/Selmer.lean |
1 |
3 |
['AntoineChambert-Loir', 'github-actions'] |
nobody |
0-38933 10 hours ago |
62-37822 2 months ago |
0-1 1 second |
28477 |
yapudpill author:yapudpill |
feat(RingTheory): golf `IsPrincipalIdealRing.of_prime` |
In complement to #28451 and as discussed in #27200, this PR uses the newly added Oka predicates to golf the proof of `IsPrincipalIdealRing.of_prime`.
---
- [x] depends on: #28525
- [x] depends on: #29567
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
new-contributor
|
53/55 |
Mathlib/RingTheory/PrincipalIdealDomain.lean,Mathlib/RingTheory/PrincipalIdealDomainOfPrime.lean |
2 |
11 |
['Ruben-VandeVelde', 'github-actions', 'kckennylau', 'mathlib4-dependent-issues-bot', 'yapudpill'] |
nobody |
0-38202 10 hours ago |
0-38202 10 hours ago |
6-28518 6 days |
28451 |
yapudpill author:yapudpill |
feat(RingTheory/Noetherian): add `IsNoetherianRing.of_prime` |
This PR introduces the first usage of `Ideal.IsOka` introduced in #27200 to prove that if all prime ideals of a `CommRing` are finitely generated then this ring is Noetherian.
To do so, we also added the lemma `Ideal.mem_span_range_self`.
---
- [x] depends on: #28525
- [x] depends on: #29567
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
new-contributor
awaiting-author
|
100/29 |
Mathlib.lean,Mathlib/RingTheory/Ideal/Span.lean,Mathlib/RingTheory/Noetherian/OfPrime.lean,docs/references.bib |
4 |
11 |
['github-actions', 'kckennylau', 'mathlib4-dependent-issues-bot', 'yapudpill'] |
nobody |
0-35031 9 hours ago |
0-54567 15 hours ago |
6-62492 6 days |
28061 |
CoolRmal author:CoolRmal |
feat(MeasureTheory): Uniqueness of Measures in the Riesz–Markov–Kakutani Representation Theorem |
This PR adds the proof of the uniqueness of measures in the Riesz–Markov–Kakutani representation theorem (i.e. if two regular measures on a locally compact Hausdorff space induce the same linear functionals on the set of compactly supported continuous functions, then these two measures are equal).
cf. https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Uniqueness.20in.20Riesz.E2.80.93Markov.E2.80.93Kakutani.20representation.20theorem
---
- [ ] depends on: #28059
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-measure-probability
|
182/0 |
Mathlib/MeasureTheory/Integral/RieszMarkovKakutani/NNReal.lean,Mathlib/MeasureTheory/Integral/RieszMarkovKakutani/Real.lean,Mathlib/MeasureTheory/Measure/Regular.lean,Mathlib/Topology/UrysohnsLemma.lean |
4 |
12 |
['CoolRmal', 'github-actions', 'j-loreaux', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
RemyDegenne assignee:RemyDegenne |
0-34930 9 hours ago |
7-37675 7 days ago |
7-43246 7 days |
28695 |
chrisflav author:chrisflav |
feat(RingTheory): meta properties of bijective ring homomorphisms |
In particular, we show that bijective is a property local on the (algebraic) source.
---
- [x] depends on: #28642
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
large-import
|
170/7 |
Mathlib.lean,Mathlib/Algebra/Algebra/Basic.lean,Mathlib/Algebra/Algebra/Hom.lean,Mathlib/LinearAlgebra/TensorProduct/Basic.lean,Mathlib/RingTheory/LocalProperties/Exactness.lean,Mathlib/RingTheory/LocalRing/ResidueField/Instances.lean,Mathlib/RingTheory/Localization/Algebra.lean,Mathlib/RingTheory/Localization/Away/Basic.lean,Mathlib/RingTheory/Localization/Basic.lean,Mathlib/RingTheory/RingHom/Bijective.lean,Mathlib/RingTheory/TensorProduct/Basic.lean |
11 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
kbuzzard assignee:kbuzzard |
0-34929 9 hours ago |
10-54588 10 days ago |
10-57634 10 days |
29322 |
xroblot author:xroblot |
feat(RingTheory/Localization/AtPrime): bijection between prime ideals |
Let `R ⊆ S` be an extension of rings and `p` be a prime ideal of `R`. Denote by `Rₚ` the localization of `R` at the complement of `p` and by `Sₚ` the localization of `S` at the (image) of the complement of `p`.
In this PR, we study the extension `Rₚ ⊆ Sₚ` and the relation between the (nonzero) prime ideals of `Sₚ` and the prime ideals of `S` above `p`. In particular, we prove that (under suitable conditions) they are in bijection. In a following PR #27706, we prove that the residual degree and ramification index are preserved by this bijection.
Note. The new file `RingTheory.Localization.AtPrime.Extension` is imported in `RingTheory.Trace.Quotient` because one function from the latter was moved to the former, but the plan is eventually to move the isomorphisms proved in `RingTheory.Trace.Quotient` to `RingTheory.Localization.AtPrime.Basic` and `RingTheory.Localization.AtPrime.Extension` where they belong. This will be done in #27706.
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory |
145/8 |
Mathlib.lean,Mathlib/RingTheory/DedekindDomain/Instances.lean,Mathlib/RingTheory/Ideal/Maps.lean,Mathlib/RingTheory/Ideal/Over.lean,Mathlib/RingTheory/Localization/AtPrime/Extension.lean,Mathlib/RingTheory/Trace/Quotient.lean |
6 |
1 |
['github-actions'] |
chrisflav assignee:chrisflav |
0-34928 9 hours ago |
9-67044 9 days ago |
9-67084 9 days |
29330 |
plp127 author:plp127 |
chore: define `Fin.cycleIcc` with conditions |
Redefine `Fin.cycleIcc` using conditionals instead of composing existing `Fin` operations together. Its worst-case runtime drops from O(n) to O(1). As a bonus, the definition no longer needs explaining.
---
[](https://gitpod.io/from-referrer/)
|
t-group-theory |
67/68 |
Mathlib/GroupTheory/Perm/Fin.lean |
1 |
7 |
['JovanGerb', 'eric-wieser', 'github-actions', 'plp127', 'tb65536'] |
tb65536 assignee:tb65536 |
0-34928 9 hours ago |
9-50554 9 days ago |
9-50591 9 days |
29341 |
joelriou author:joelriou |
feat(Topology): the topology generated by a family of spaces |
Some categories of topological spaces are "convenient" in the sense that they have nice categorical properties (e.g. they have limits, colimits and are cartesian closed). This PR is the first in a series towards showing that delta generated spaces form a cartesian closed monoidal category (see https://github.com/joelriou/topcat-model-category/blob/852a514c1d955ab586507bcd5a7b5efb99c6c3df/TopCatModelCategory/Convenient/CartesianClosed.lean#L92 for the general result), and this result is part of my formalization effort towards the Quillen model category structure on simplicial sets.
In this PR, given a family `X` of topological spaces, and a topological space `Y`, we introduce the `X`-generated topology on `Y`, which is coinduced by all continuous maps `X i → Y`.
(Eventually, this will generalize previous works by Dagur Asgeirsson and Ben Eltschig about compactly/delta generated spaces in mathlib. At some point, their definitions will be refactored as particular cases of the definitions in this PR series.)
---
[](https://gitpod.io/from-referrer/)
|
t-topology |
241/0 |
Mathlib.lean,Mathlib/Topology/Convenient/GeneratedBy.lean,docs/references.bib |
3 |
1 |
['github-actions'] |
jcommelin assignee:jcommelin |
0-34927 9 hours ago |
9-4162 9 days ago |
9-4143 9 days |
29361 |
FlAmmmmING author:FlAmmmmING |
feat(RingTheory/PowerSeries/Catalan.lean) |
We introduce the Catalan generating function as a formal power series over `ℕ`.
## Main Definitions
* `PowerSeries.catalanSeries`: The Catalan generating function as a power series.
## Main Results
* `PowerSeries.sum_coeff_X_catalanSeries`: When `n` is a natural number,
each term in the sum `coeff i X * catalan (n - i)` is 0 except for `i = 1`.
* `PowerSeries.coeff_X_mul_catalanSeries`: The coefficient of `X * catalanSeries` at `X^n` is
`catalan (n - 1)` when `n > 0`.
* `PowerSeries.catalanSeries_one_add_X_mul_self_sq`: The Catalan generating function satisfies the
equation `catalanSeries = 1 + X * catalanSeries ^ 2`.
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
new-contributor
|
89/0 |
Mathlib.lean,Mathlib/RingTheory/PowerSeries/Catalan.lean |
2 |
2 |
['github-actions', 'wwylele'] |
kbuzzard assignee:kbuzzard |
0-34926 9 hours ago |
8-7589 8 days ago |
8-7624 8 days |
29588 |
Periecle author:Periecle |
feat(Analysis/Complex/Residue): Implement residue theory for complex functions at isolated singularities |
# Add basic residue theory for complex functions
This PR introduces the residue theory implementation in mathlib.
## Main additions
- **`HasIsolatedSingularityAt f c`**: Predicate for functions with isolated singularities at point `c`
- **`residue f c hf`**: The residue of `f` at isolated singularity `c`, defined via circle integrals
- **Radius independence**: `residue_eq_two_pi_I_inv_smul_circleIntegral` - residue equals normalized circle integral for any valid radius
- **Holomorphic residues**: `residue_of_holomorphic` - functions holomorphic in a neighborhood have zero residue
- **Simple pole formula**: `residue_simple_pole` - for `f(z) = (z-c)⁻¹ * g(z)`, residue equals `g(c)`
## Implementation notes
- Builds on existing circle integral infrastructure in `CauchyIntegral.lean`
- Uses `Classical.choose` to extract witness radius from isolated singularity condition
- Comprehensive documentation with mathematical context and examples
- Establishes foundation for residue theorem, argument principle, and other applications
## Examples included
- `residue(1/z, 0) = 1` (canonical simple pole)
- Radius independence demonstration
- Zero residues for holomorphic functions
This provides the essential building blocks for complex analysis and first step to formalize residue theory. |
new-contributor
t-analysis
|
383/0 |
Mathlib/Analysis/Complex/Residue/Basic.lean |
1 |
2 |
['github-actions', 'llllvvuu'] |
nobody |
0-32263 8 hours ago |
0-80468 22 hours ago |
0-80504 22 hours |
29208 |
ShreckYe author:ShreckYe |
feat(Algebra/GCDMonoid/Finset): change the signature of `lcm_eq_zero_iff` to its simp normal form and add `lcm_ne_zero_iff` theorems |
This PR is similar to #28897 and I found a need for one of the added theorems in #29204.
I've noticed that the existing theorem `lcm_eq_zero_iff`'s rhs term `0 ∈ f '' s` is not in simp normal form. Should this be deprecated and replaced? I have left comments about this in the code. |
t-algebra
delegated
label:t-algebra$ |
11/4 |
Mathlib/Algebra/GCDMonoid/Finset.lean,Mathlib/Algebra/GCDMonoid/Multiset.lean |
2 |
14 |
['Ruben-VandeVelde', 'ShreckYe', 'github-actions', 'mathlib-bors', 'ocfnash'] |
ocfnash assignee:ocfnash |
0-26060 7 hours ago |
0-66719 18 hours ago |
10-24094 10 days |
29611 |
vihdzp author:vihdzp |
feat: alternate characterization of `≤` on Archimedean classes |
The definition of `mk x ≤ mk y` is that `|y| ≤ n * |x|` for some natural `n`. We prove the alternate characterization that `q * |y| ≤ |x|` for some positive rational `q`, and in fact prove a more general version for any densely ordered ring.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
37/1 |
Mathlib/Algebra/Order/Ring/Archimedean.lean |
1 |
1 |
['github-actions'] |
nobody |
0-26053 7 hours ago |
0-26149 7 hours ago |
0-26191 7 hours |
27936 |
alreadydone author:alreadydone |
feat(Algebra): additivize Dvd and Prime |
`Prime` can't be directly additivized, so we introduce `Preprime`, which drops the `≠ 0` condition, and additivize it to `AddPrime`. To show that `Preprime` is a reasonable definition, we show its connection to `Irreducible` under `IsPrimal` and `IsRegular` conditions. We also show that an element in a product monoid is preprime iff one component is a unit and the other is preprime, and the same with `Preprime` replaced by `Irreducible`.
Also additivize `IsPrimal`, `IsRelPrime` and `DecompositionMonoid`.
The motivation is that the primality of `single g 1` in `AddMonoidAlgebra k G` is connected to the primality of `g` in `G`.
---
I've checked [all 29 files](https://github.com/search?q=repo%3Aleanprover-community%2Fmathlib4%20%E2%88%A3%20to_additive&type=code) containing the `∣` symbol and the `to_additive` attribute and fixed the wrongly translated (`dvd` to `addDvd`) names.
TODO: connect (Add)Dvd to [ExistsMul/AddOfLE](https://leanprover-community.github.io/mathlib4_docs/Mathlib/Algebra/Order/Monoid/Unbundled/ExistsOfLE.html#ExistsMulOfLE)
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
400/191 |
Mathlib.lean,Mathlib/Algebra/BigOperators/Group/Finset/Basic.lean,Mathlib/Algebra/BigOperators/Group/Finset/Defs.lean,Mathlib/Algebra/BigOperators/Group/Finset/Piecewise.lean,Mathlib/Algebra/BigOperators/Group/List/Lemmas.lean,Mathlib/Algebra/BigOperators/Group/Multiset/Basic.lean,Mathlib/Algebra/Divisibility/Basic.lean,Mathlib/Algebra/Divisibility/Finite.lean,Mathlib/Algebra/Divisibility/Hom.lean,Mathlib/Algebra/Divisibility/Prod.lean,Mathlib/Algebra/Divisibility/Units.lean,Mathlib/Algebra/Group/Action/Pointwise/Finset.lean,Mathlib/Algebra/Group/Prod.lean,Mathlib/Algebra/GroupWithZero/Associated.lean,Mathlib/Algebra/Notation/Defs.lean,Mathlib/Algebra/Prime/Defs.lean,Mathlib/Algebra/Prime/Lemmas.lean,Mathlib/Algebra/Prime/Prod.lean,Mathlib/Data/Nat/Prime/Defs.lean,Mathlib/Dynamics/PeriodicPts/Defs.lean,Mathlib/GroupTheory/Coset/Card.lean,Mathlib/GroupTheory/Exponent.lean,Mathlib/GroupTheory/GroupAction/Blocks.lean,Mathlib/GroupTheory/GroupAction/Period.lean,Mathlib/GroupTheory/Index.lean,Mathlib/GroupTheory/OrderOfElement.lean,Mathlib/GroupTheory/Perm/Cycle/Type.lean,Mathlib/GroupTheory/Schreier.lean,Mathlib/GroupTheory/SpecificGroups/Cyclic.lean,Mathlib/Tactic/ToAdditive/GuessName.lean |
30 |
9 |
['JovanGerb', 'adomani', 'alreadydone', 'bryangingechen', 'github-actions', 'mathlib4-merge-conflict-bot'] |
bryangingechen assignee:bryangingechen |
0-24964 6 hours ago |
7-45992 7 days ago |
38-21555 38 days |
29354 |
themathqueen author:themathqueen |
refactor(Algebra/Algebra/Equiv): allow for non-unital `AlgEquiv` |
This refactors `AlgEquiv` to allow for non-unital algebras. More specifically, we weaken the type class assumptions from:
```lean
structure AlgEquiv (R A B : Type*) [CommSemiring R] [Semiring A] [Semiring B]
[Algebra R A] [Algebra R B]
```
to
```lean
structure AlgEquiv (R A B : Type*) [Add A] [Add B] [Mul A] [Mul B]
[SMul R A] [SMul R B]
```
Instead of a `commutes'` field, we now have a `map_smul'` field. We also include a definition `AlgEquiv.ofCommutes` which takes in a `RingEquiv` and a `commutes'` field to match before and for convenience.
Co-authored-by: Jireh Loreaux
---
Revives #8686.
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
471/399 |
Mathlib/Algebra/Algebra/Equiv.lean,Mathlib/Algebra/Algebra/Opposite.lean,Mathlib/Algebra/Algebra/Pi.lean,Mathlib/Algebra/Algebra/Prod.lean,Mathlib/Algebra/Algebra/Subalgebra/Basic.lean,Mathlib/Algebra/Algebra/Subalgebra/MulOpposite.lean,Mathlib/Algebra/Algebra/Tower.lean,Mathlib/Algebra/Algebra/TransferInstance.lean,Mathlib/Algebra/Category/AlgCat/Basic.lean,Mathlib/Algebra/Category/CommAlgCat/Basic.lean,Mathlib/Algebra/Category/CommAlgCat/FiniteType.lean,Mathlib/Algebra/Category/Ring/Constructions.lean,Mathlib/Algebra/DualQuaternion.lean,Mathlib/Algebra/MonoidAlgebra/Basic.lean,Mathlib/Algebra/MonoidAlgebra/ToDirectSum.lean,Mathlib/Algebra/MvPolynomial/Equiv.lean,Mathlib/Algebra/MvPolynomial/Rename.lean,Mathlib/Algebra/Polynomial/AlgebraMap.lean,Mathlib/Algebra/Polynomial/Taylor.lean,Mathlib/Algebra/Quaternion.lean,Mathlib/Algebra/Star/Free.lean,Mathlib/Algebra/Star/StarAlgHom.lean,Mathlib/Analysis/Normed/Algebra/Spectrum.lean,Mathlib/Analysis/Normed/Algebra/UnitizationL1.lean,Mathlib/Analysis/Normed/Lp/LpEquiv.lean,Mathlib/Analysis/RCLike/Basic.lean,Mathlib/Data/Matrix/Basic.lean,Mathlib/Data/Matrix/Composition.lean,Mathlib/Data/Matrix/DualNumber.lean,Mathlib/FieldTheory/Fixed.lean,Mathlib/FieldTheory/Galois/Basic.lean,Mathlib/FieldTheory/Galois/Profinite.lean,Mathlib/FieldTheory/IntermediateField/Adjoin/Basic.lean,Mathlib/FieldTheory/IntermediateField/Basic.lean,Mathlib/FieldTheory/Normal/Basic.lean,Mathlib/FieldTheory/PrimitiveElement.lean,Mathlib/FieldTheory/RatFunc/Basic.lean,Mathlib/FieldTheory/Separable.lean,Mathlib/LinearAlgebra/CliffordAlgebra/BaseChange.lean,Mathlib/LinearAlgebra/CliffordAlgebra/Conjugation.lean,Mathlib/LinearAlgebra/Complex/Module.lean,Mathlib/LinearAlgebra/Matrix/Basis.lean,Mathlib/LinearAlgebra/Matrix/Charpoly/Coeff.lean,Mathlib/LinearAlgebra/Matrix/Charpoly/LinearMap.lean,Mathlib/LinearAlgebra/Matrix/Reindex.lean,Mathlib/LinearAlgebra/Matrix/ToLin.lean,Mathlib/LinearAlgebra/Matrix/Unique.lean,Mathlib/LinearAlgebra/TensorProduct/Graded/Internal.lean,Mathlib/RingTheory/AdjoinRoot.lean,Mathlib/RingTheory/Bialgebra/Equiv.lean,Mathlib/RingTheory/DedekindDomain/Different.lean,Mathlib/RingTheory/Etale/Field.lean,Mathlib/RingTheory/Finiteness/Basic.lean,Mathlib/RingTheory/Flat/Equalizer.lean,Mathlib/RingTheory/FractionalIdeal/Operations.lean,Mathlib/RingTheory/Frobenius.lean,Mathlib/RingTheory/GradedAlgebra/Basic.lean,Mathlib/RingTheory/HahnSeries/PowerSeries.lean,Mathlib/RingTheory/Ideal/Operations.lean,Mathlib/RingTheory/Ideal/Over.lean,Mathlib/RingTheory/Ideal/Quotient/Operations.lean,Mathlib/RingTheory/IntegralClosure/IntegrallyClosed.lean,Mathlib/RingTheory/Invariant/Basic.lean,Mathlib/RingTheory/Invariant/Profinite.lean,Mathlib/RingTheory/IsTensorProduct.lean,Mathlib/RingTheory/Jacobson/Artinian.lean,Mathlib/RingTheory/Jacobson/Ring.lean,Mathlib/RingTheory/Kaehler/Basic.lean,Mathlib/RingTheory/LaurentSeries.lean,Mathlib/RingTheory/Localization/Basic.lean,Mathlib/RingTheory/Localization/FractionRing.lean,Mathlib/RingTheory/MatrixAlgebra.lean,Mathlib/RingTheory/MvPolynomial/Localization.lean,Mathlib/RingTheory/Norm/Basic.lean,Mathlib/RingTheory/Polynomial/Quotient.lean,Mathlib/RingTheory/PolynomialAlgebra.lean,Mathlib/RingTheory/PowerSeries/WeierstrassPreparation.lean,Mathlib/RingTheory/RingHom/FiniteType.lean,Mathlib/RingTheory/SimpleModule/Isotypic.lean,Mathlib/RingTheory/Smooth/Basic.lean,Mathlib/RingTheory/Smooth/Pi.lean,Mathlib/RingTheory/Spectrum/Prime/Polynomial.lean,Mathlib/RingTheory/TensorProduct/Basic.lean,Mathlib/RingTheory/TensorProduct/MvPolynomial.lean,Mathlib/RingTheory/TensorProduct/Pi.lean,Mathlib/RingTheory/TensorProduct/Quotient.lean,Mathlib/RingTheory/Trace/Basic.lean,Mathlib/RingTheory/Unramified/Field.lean,Mathlib/Topology/Algebra/Algebra/Equiv.lean,Mathlib/Topology/Algebra/Module/FiniteDimension.lean,Mathlib/Topology/LocallyConstant/Algebra.lean |
91 |
10 |
['github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'mathlib4-merge-conflict-bot', 'themathqueen'] |
nobody |
0-22044 6 hours ago |
0-22044 6 hours ago |
0-41545 11 hours |
26920 |
yuma-mizuno author:yuma-mizuno |
feat(Tactic.CategoryTheory): add associator inserting tactic |
---
[](https://gitpod.io/from-referrer/)
|
t-category-theory
t-meta
WIP
|
714/0 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/CategoryTheory/Associators.lean,MathlibTest/CategoryTheory/Associators.lean |
4 |
1 |
['github-actions'] |
nobody |
0-18825 5 hours ago |
66-12600 2 months ago |
0-16 16 seconds |
29558 |
Thmoas-Guan author:Thmoas-Guan |
feat(Algebra): definition of global dimension |
In this PR, we define projective dimension and global dimension using `CategoryTheory.HasProjectiveDimensionLT`
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
WIP
|
73/0 |
Mathlib.lean,Mathlib/RingTheory/GlobalDimension.lean |
2 |
1 |
['github-actions'] |
nobody |
0-17628 4 hours ago |
0-17628 4 hours ago |
0-0 0 seconds |
26601 |
yuma-mizuno author:yuma-mizuno |
feat(CategoryTheory): make `Functor.comp` irreducible |
[#mathlib4 > Functor identity `𝟭 _ ⋙ F = F` is definitional equality](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Functor.20identity.20.60.F0.9D.9F.AD.20_.20.E2.8B.99.20F.20.3D.20F.60.20is.20definitional.20equality/with/523978659)
---
[](https://gitpod.io/from-referrer/)
|
t-category-theory
WIP
|
514/261 |
Mathlib/AlgebraicTopology/DoldKan/Compatibility.lean,Mathlib/AlgebraicTopology/SimplexCategory/Defs.lean,Mathlib/CategoryTheory/Adjunction/Basic.lean,Mathlib/CategoryTheory/CatCommSq.lean,Mathlib/CategoryTheory/Category/Cat.lean,Mathlib/CategoryTheory/Category/RelCat.lean,Mathlib/CategoryTheory/Category/ULift.lean,Mathlib/CategoryTheory/Core.lean,Mathlib/CategoryTheory/Discrete/Basic.lean,Mathlib/CategoryTheory/EqToHom.lean,Mathlib/CategoryTheory/Equivalence.lean,Mathlib/CategoryTheory/Functor/Basic.lean,Mathlib/CategoryTheory/Functor/Category.lean,Mathlib/CategoryTheory/Functor/Const.lean,Mathlib/CategoryTheory/Functor/Currying.lean,Mathlib/CategoryTheory/Functor/CurryingThree.lean,Mathlib/CategoryTheory/Functor/FullyFaithful.lean,Mathlib/CategoryTheory/Functor/Functorial.lean,Mathlib/CategoryTheory/Functor/ReflectsIso/Basic.lean,Mathlib/CategoryTheory/Functor/TwoSquare.lean,Mathlib/CategoryTheory/Groupoid/FreeGroupoid.lean,Mathlib/CategoryTheory/Join/Basic.lean,Mathlib/CategoryTheory/Limits/Cones.lean,Mathlib/CategoryTheory/Limits/Shapes/Pullback/Categorical/Basic.lean,Mathlib/CategoryTheory/ObjectProperty/FullSubcategory.lean,Mathlib/CategoryTheory/Opposites.lean,Mathlib/CategoryTheory/PathCategory/Basic.lean,Mathlib/CategoryTheory/Pi/Basic.lean,Mathlib/CategoryTheory/Products/Associator.lean,Mathlib/CategoryTheory/Products/Basic.lean,Mathlib/CategoryTheory/Quotient.lean,Mathlib/CategoryTheory/Sigma/Basic.lean,Mathlib/CategoryTheory/Whiskering.lean,Mathlib/CategoryTheory/Yoneda.lean |
34 |
2 |
['github-actions', 'leanprover-community-bot-assistant'] |
nobody |
0-16678 4 hours ago |
0-17640 4 hours ago |
0-10 10 seconds |
29613 |
RemyDegenne author:RemyDegenne |
chore(Probability): rename IsFiniteKernel.bound to Kernel.bound |
That definition was specific to finite kernels before #29137, but not anymore. Also the new name allows dot notation.
---
[](https://gitpod.io/from-referrer/)
|
t-measure-probability |
73/61 |
Mathlib/Probability/Kernel/Basic.lean,Mathlib/Probability/Kernel/Composition/Comp.lean,Mathlib/Probability/Kernel/Composition/CompProd.lean,Mathlib/Probability/Kernel/Composition/MapComap.lean,Mathlib/Probability/Kernel/Composition/ParallelComp.lean,Mathlib/Probability/Kernel/Defs.lean,Mathlib/Probability/Kernel/Integral.lean,Mathlib/Probability/Kernel/RadonNikodym.lean,Mathlib/Probability/Kernel/WithDensity.lean |
9 |
1 |
['github-actions'] |
nobody |
0-14332 3 hours ago |
0-14409 3 hours ago |
0-14447 4 hours |
29610 |
llllvvuu author:llllvvuu |
feat(LinearAlgebra): define LinearMap.Diagonalization |
---
[](https://gitpod.io/from-referrer/)
|
|
89/0 |
Mathlib/junk.lean |
1 |
1 |
['github-actions'] |
nobody |
0-13280 3 hours ago |
0-27807 7 hours ago |
0-0 0 seconds |
29604 |
mans0954 author:mans0954 |
refactor(Analysis/LocallyConvex/WithSeminorms): Relax some of the hypothesis |
Relax some of the hypothesis in `Analysis/LocallyConvex/WithSeminorms`
---
[](https://gitpod.io/from-referrer/)
|
t-analysis |
33/22 |
Mathlib/Analysis/LocallyConvex/WithSeminorms.lean |
1 |
1 |
['github-actions'] |
nobody |
0-10668 2 hours ago |
0-54324 15 hours ago |
0-54362 15 hours |
28846 |
euprunin author:euprunin |
chore(RingTheory/HahnSeries): golf entire `C_ne_zero` using `grind` |
---
Show trace profiling of C_ne_zero : <10 ms before, 53 ms after
### Trace profiling of `C_ne_zero` before PR 28846
```diff
diff --git a/Mathlib/RingTheory/HahnSeries/Multiplication.lean b/Mathlib/RingTheory/HahnSeries/Multiplication.lean
index 28af8d93db..e397a14bce 100644
--- a/Mathlib/RingTheory/HahnSeries/Multiplication.lean
+++ b/Mathlib/RingTheory/HahnSeries/Multiplication.lean
@@ -768,6 +768,7 @@ theorem C_injective : Function.Injective (C : R → HahnSeries Γ R) := by
have h := rs 0
rwa [C_apply, coeff_single_same, C_apply, coeff_single_same] at h
+set_option trace.profiler true in
theorem C_ne_zero {r : R} (h : r ≠ 0) : (C r : HahnSeries Γ R) ≠ 0 := by
contrapose! h
rw [← C_zero] at h
```
```
✔ [1128/1128] Built Mathlib.RingTheory.HahnSeries.Multiplication (3.8s)
Build completed successfully (1128 jobs).
```
### Trace profiling of `C_ne_zero` after PR 28846
```diff
diff --git a/Mathlib/RingTheory/HahnSeries/Multiplication.lean b/Mathlib/RingTheory/HahnSeries/Multiplication.lean
index 28af8d93db..0095b92923 100644
--- a/Mathlib/RingTheory/HahnSeries/Multiplication.lean
+++ b/Mathlib/RingTheory/HahnSeries/Multiplication.lean
@@ -768,10 +768,9 @@ theorem C_injective : Function.Injective (C : R → HahnSeries Γ R) := by
have h := rs 0
rwa [C_apply, coeff_single_same, C_apply, coeff_single_same] at h
+set_option trace.profiler true in
theorem C_ne_zero {r : R} (h : r ≠ 0) : (C r : HahnSeries Γ R) ≠ 0 := by
- contrapose! h
- rw [← C_zero] at h
- exact C_injective h
+ grind [C_apply, single_eq_zero_iff]
theorem order_C {r : R} : order (C r : HahnSeries Γ R) = 0 := by
by_cases h : r = 0
```
```
ℹ [1128/1128] Built Mathlib.RingTheory.HahnSeries.Multiplication (3.8s)
info: Mathlib/RingTheory/HahnSeries/Multiplication.lean:772:0: [Elab.async] [0.053582] elaborating proof of HahnSeries.C_ne_zero
[Elab.definition.value] [0.053275] HahnSeries.C_ne_zero
[Elab.step] [0.053120] grind [C_apply, single_eq_zero_iff]
[Elab.step] [0.053115] grind [C_apply, single_eq_zero_iff]
[Elab.step] [0.053107] grind [C_apply, single_eq_zero_iff]
[Meta.synthInstance] [0.015414] ❌️ Lean.Grind.IntModule (HahnSeries Γ R)
Build completed successfully (1128 jobs).
```
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
awaiting-author
|
1/3 |
Mathlib/RingTheory/HahnSeries/Multiplication.lean |
1 |
10 |
['Ruben-VandeVelde', 'euprunin', 'github-actions', 'grunweg', 'leanprover-bot', 'leanprover-community-mathlib4-bot'] |
chrisflav assignee:chrisflav |
0-9409 2 hours ago |
0-9409 2 hours ago |
11-49867 11 days |
28612 |
euprunin author:euprunin |
chore(Data/List): golf entire `idxOf_append_of_mem`, `cons_sublist_cons'`, `length_eraseIdx_add_one`, `length_eraseP_add_one` and `idxOf_append_of_notMem` using `grind` |
---
[](https://gitpod.io/from-referrer/)
|
t-data
maintainer-merge
|
5/26 |
Mathlib/Data/List/Basic.lean |
1 |
7 |
['euprunin', 'github-actions', 'grunweg', 'leanprover-bot', 'leanprover-community-mathlib4-bot'] |
nobody |
0-9290 2 hours ago |
0-9290 2 hours ago |
16-67738 16 days |
27107 |
AntoineChambert-Loir author:AntoineChambert-Loir |
feat(GroupTheory/GroupAction/SubMulAction/Combination) : combinations and group actions |
`Nat.Combination X n` is the type all `s : Finset X` such that `s.card = n`.
This PR provides some API for this subtype and the `SubMulAction` it inherits when a group acts on `X`.
It will be used in conjunction with the description of some maximal subgroups of `Equiv.Perm X` to construct primitive actions.
Question on the names: when `X` is a fintype, there is `Finset.powersetCard` that gives the same object, as a `Finset`. But the present PR also applies when `X` is infinite. Then maybe `Nat.Combination` should be renamed as `Set.powersetCard`?
---
[](https://gitpod.io/from-referrer/)
|
t-group-theory |
324/0 |
Mathlib.lean,Mathlib/Data/Fintype/EquivFin.lean,Mathlib/Data/Nat/Choose/Basic.lean,Mathlib/GroupTheory/GroupAction/SubMulAction/Combination.lean |
4 |
39 |
['AntoineChambert-Loir', 'alreadydone', 'github-actions', 'tb65536'] |
alreadydone assignee:alreadydone |
0-8151 2 hours ago |
39-3351 1 month ago |
61-33096 61 days |
27400 |
dleijnse author:dleijnse |
feat: define geometrically reduced algebras |
Define geometrically reduced algebras, and prove that if all finitely generated subalgebras of an algebra `A` are geometrically reduced, then `A` is geometrically reduced.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-algebra
label:t-algebra$ |
105/0 |
Mathlib.lean,Mathlib/RingTheory/Adjoin/FG.lean,Mathlib/RingTheory/Nilpotent/Defs.lean,Mathlib/RingTheory/Nilpotent/GeometricallyReduced.lean,Mathlib/RingTheory/TensorProduct/Basic.lean |
5 |
48 |
['dleijnse', 'github-actions', 'joelriou', 'kckennylau'] |
joelriou assignee:joelriou |
0-6614 1 hour ago |
2-11058 2 days ago |
48-77114 48 days |
29603 |
gasparattila author:gasparattila |
feat(Algebra/AddTorsor/Basic): add `Pi.vsub_apply` |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
easy
label:t-algebra$ |
9/1 |
Mathlib/Algebra/AddTorsor/Basic.lean |
1 |
5 |
['eric-wieser', 'gasparattila', 'github-actions'] |
nobody |
0-2704 45 minutes ago |
0-59420 16 hours ago |
0-59458 16 hours |
29327 |
loefflerd author:loefflerd |
feat(NumberTheory/ModularForms): Cusps of subgroups acting on upper half-plane |
- Define "arithmetic subgroups" of GL(2, R), as subgroups commensurable with the image of SL(2, Z)
- Add some notations and API to make it easier to work with images in GL(2, R) of subgroups of SL(2, Z)
- Define "cusps" of a subgroup of GL(2, R), as fixed points of parabolic elements on P^1(R).
- Prove that the cusps of an arithmetic subgroup are precisely P^1(Q).
---
Carved off from the larger WIP PR #26651
|
t-number-theory |
256/33 |
Mathlib.lean,Mathlib/LinearAlgebra/Matrix/GeneralLinearGroup/Defs.lean,Mathlib/NumberTheory/ModularForms/ArithmeticSubgroups.lean,Mathlib/NumberTheory/ModularForms/CongruenceSubgroups.lean,Mathlib/NumberTheory/ModularForms/Cusps.lean,Mathlib/NumberTheory/ModularForms/SlashInvariantForms.lean |
6 |
29 |
['CBirkbeck', 'github-actions', 'loefflerd', 'riccardobrasca'] |
riccardobrasca assignee:riccardobrasca |
0-2685 44 minutes ago |
8-79688 8 days ago |
9-55291 9 days |
27599 |
mitchell-horner author:mitchell-horner |
feat(Combinatorics/SimpleGraph): define `CompleteEquipartiteSubgraph` |
Define the complete equipartite subgraphs in `r` parts each of size `t` in `G` as the `r` subsets of vertices each of size `t` such that vertices in distinct subsets are adjacent.
In this case `Nonempty (G.CompleteEquipartiteSubgraph r t)` is equivalent to `completeEquipartiteGraph r t ⊑ G`, that is, finding `r` subsets of vertices each of size `t` in `G` such that vertices in distinct subsets are adjacent is equivalent to finding an injective homomorphism from `completeEquipartiteGraph r t` to `G`.
---
- [x] depends on: #27597
[](https://gitpod.io/from-referrer/)
|
t-combinatorics |
113/7 |
Mathlib/Combinatorics/SimpleGraph/CompleteMultipartite.lean |
1 |
19 |
['YaelDillies', 'b-mehta', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'mitchell-horner'] |
YaelDillies assignee:YaelDillies |
0-2019 33 minutes ago |
9-70681 9 days ago |
18-28023 18 days |
29615 |
eric-wieser author:eric-wieser |
chore: add a computable shortcut for `AddCommMonoid ℂ` |
---
[](https://gitpod.io/from-referrer/)
|
bench-after-CI
t-analysis
easy
|
9/1 |
Mathlib/Analysis/Complex/Basic.lean |
1 |
1 |
['github-actions'] |
nobody |
0-1731 28 minutes ago |
0-1801 29 minutes ago |
0-1795 29 minutes |
28862 |
edegeltje author:edegeltje |
feat(TacticAnalysis): add a linter for merging consequent intro tactics |
The linter is triggered by setting the option `linter.tacticAnalysis.introMerge` (which is on by default).
When it finds consequent `intro` tactics, it will give a warning suggesting a single use of `intro`.
For example:
```lean4
set_option linter.tacticAnalysis.introMerge true
/-- warning: Try this: intro a b -/
#guard_msgs in
example : ∀ a b : Unit, a = b := by
intro a
intro b
rfl
```
---
[](https://gitpod.io/from-referrer/)
|
t-meta
delegated
|
73/23 |
Mathlib/CategoryTheory/Idempotents/Basic.lean,Mathlib/CategoryTheory/Limits/MonoCoprod.lean,Mathlib/CategoryTheory/Sites/Coverage.lean,Mathlib/Data/PNat/Prime.lean,Mathlib/Data/QPF/Multivariate/Constructions/Fix.lean,Mathlib/Order/Category/NonemptyFinLinOrd.lean,Mathlib/Order/OmegaCompletePartialOrder.lean,Mathlib/RingTheory/RootsOfUnity/Minpoly.lean,Mathlib/Tactic/TacticAnalysis/Declarations.lean,MathlibTest/TacticAnalysis.lean,MathlibTest/success_if_fail_with_msg.lean |
11 |
18 |
['Vierkantor', 'edegeltje', 'euprunin', 'github-actions', 'grunweg', 'mathlib-bors', 'thorimur'] |
dwrensha assignee:dwrensha |
0-1576 26 minutes ago |
0-73262 20 hours ago |
18-79642 18 days |
27602 |
mitchell-horner author:mitchell-horner |
feat(Combinatorics/SimpleGraph): define `CompleteBipartiteSubgraph` |
Define the complete bipartite subgraphs of `s` and `t` parts as a "left" subset of `s` vertices and a "right" subset of `t` vertices such that every vertex in the "left" subset is adjacent to every vertex in the "right" subset.
In this case `Nonempty (G.CompleteBipartiteSubgraph (card α) (card β))` is equivalent to `completeBipartiteGraph α β ⊑ G`, that is, finding a "left" subset of `s` vertices and a "right" subset of `t` vertices such that every vertex in the "left" subset is adjacent to every vertex in the "right" subset is equivalent to finding an injective homomorphism `completeBipartiteGraph α β` to `G`.
---
[](https://gitpod.io/from-referrer/)
|
t-combinatorics |
88/0 |
Mathlib/Combinatorics/SimpleGraph/Bipartite.lean |
1 |
3 |
['github-actions', 'mitchell-horner', 'vlad902'] |
YaelDillies assignee:YaelDillies |
0-1370 22 minutes ago |
46-60904 1 month ago |
46-60952 46 days |
14426 |
adomani author:adomani |
dev: `#min_imps` command |
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict
WIP
|
142/0 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/MinImports.lean,test/MinImports.lean |
4 |
2 |
['adomani', 'github-actions'] |
nobody |
409-8945 1 year ago |
422-5326 1 year ago |
0-0 0 seconds |
14720 |
eric-wieser author:eric-wieser |
refactor: change `CliffordAlgebra.lift` to use quadratic maps |
This works towards addressing a footnote on [page 152](https://eric-wieser.github.io/thesis/eric-wieser-thesis.pdf#page=164) of my thesis.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
WIP
label:t-algebra$ |
200/167 |
Mathlib/LinearAlgebra/CliffordAlgebra/Basic.lean,Mathlib/LinearAlgebra/CliffordAlgebra/Equivs.lean,Mathlib/LinearAlgebra/CliffordAlgebra/Prod.lean,Mathlib/LinearAlgebra/QuadraticForm/Complex.lean,Mathlib/LinearAlgebra/QuadraticForm/Dual.lean,Mathlib/LinearAlgebra/QuadraticForm/Isometry.lean,Mathlib/LinearAlgebra/QuadraticForm/IsometryEquiv.lean,Mathlib/LinearAlgebra/QuadraticForm/Prod.lean,Mathlib/LinearAlgebra/QuadraticForm/QuadraticModuleCat.lean,Mathlib/LinearAlgebra/QuadraticForm/Real.lean,Mathlib/LinearAlgebra/QuadraticForm/TensorProduct/Isometries.lean |
11 |
1 |
['github-actions'] |
nobody |
409-8945 1 year ago |
422-86340 1 year ago |
0-0 0 seconds |
13847 |
alreadydone author:alreadydone |
feat(EllipticCurve): the universal elliptic curve |
+ Define the universal Weierstrass curve (`Universal.curve`) over the polynomial ring `ℤ[A₁,A₂,A₃,A₄,A₆]`, and the universal pointed elliptic curve (`Universal.pointedCurve`) over the field of fractions (`Universal.Field`) of the universal ring `ℤ[A₁,A₂,A₃,A₄,A₆,X,Y]/⟨P⟩ = Universal.Poly/⟨P⟩` (`Universal.Ring`, where `P` is the Weierstrass polynomial) with distinguished point `(X,Y)`.
+ Given a Weierstrass curve `W` over a commutative ring `R`, we define the specialization homomorphism `W.specialize : ℤ[A₁,A₂,A₃,A₄,A₆] →+* R`. If `(x,y)` is a point on the affine plane, we define `W.polyEval x y : Universal.Poly →+* R`, which factors through `W.ringEval x y : Universal.Ring →+* R` if `(x,y)` is on `W`.
+ Introduce the cusp curve `Y² = X³`, on which lies the rational point `(1,1)`, with the nice property that `ψₙ(1,1) = n`, making it easy to prove nonvanishing of the universal `ψₙ` when `n ≠ 0` by specializing to the cusp curve, which shows that `(X,Y)` is a point of infinite order on the universal pointed elliptic curve.
---
- [x] depends on: #13845
- [x] depends on: #12883
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-algebraic-geometry
merge-conflict
awaiting-author
label:t-algebra$ |
543/208 |
Mathlib.lean,Mathlib/Algebra/Polynomial/Bivariate.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Affine.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Group.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Jacobian.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Universal.lean |
6 |
4 |
['Multramate', 'alreadydone', 'github-actions', 'leanprover-community-mathlib4-bot'] |
nobody |
409-8944 1 year ago |
442-35641 1 year ago |
0-0 0 seconds |
14036 |
adomani author:adomani |
Test/decl diff in lean |
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict |
465/1040 |
.github/workflows/Lean_decl_diff.yml,.github/workflows/bors.yml,.github/workflows/build.yml,.github/workflows/build.yml.in,.github/workflows/build_fork.yml,.github/workflows/mk_build_yml.sh,scripts/decls_diff_hybrid.sh,scripts/list_decls.lean |
8 |
1 |
['github-actions'] |
nobody |
409-8944 1 year ago |
447-7235 1 year ago |
0-0 0 seconds |
14167 |
alreadydone author:alreadydone |
feat: Group scheme structure on Weierstrass curve |
---
[](https://gitpod.io/from-referrer/)
|
workshop-AIM-AG-2024
t-algebraic-geometry
merge-conflict
WIP
|
727/41 |
Mathlib.lean,Mathlib/Algebra/GroupWithZero/NonZeroDivisors.lean,Mathlib/Algebra/Polynomial/Bivariate.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Group.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Scheme.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Universal.lean,Mathlib/Data/Finsupp/Basic.lean,Mathlib/GroupTheory/MonoidLocalization.lean,Mathlib/LinearAlgebra/Basis.lean,Mathlib/LinearAlgebra/FreeModule/Basic.lean,Mathlib/RingTheory/AlgebraTower.lean,Mathlib/RingTheory/MvPolynomial/Basic.lean |
12 |
3 |
['Multramate', 'github-actions', 'jcommelin'] |
nobody |
409-8944 1 year ago |
421-82955 1 year ago |
0-0 0 seconds |
13297 |
urkud author:urkud |
feat(Semicontinuous): add `comp` lemma |
---
[](https://gitpod.io/from-referrer/) |
t-order
t-topology
merge-conflict
awaiting-author
|
31/13 |
Mathlib/Topology/Semicontinuous.lean |
1 |
3 |
['sgouezel', 'urkud'] |
nobody |
409-8943 1 year ago |
420-73074 1 year ago |
0-18175 5 hours |
13372 |
adomani author:adomani |
dev: generic replacement |
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict |
446/0 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter/ReplaceRefine.lean,Mathlib/Tactic/Replacements.lean |
4 |
4 |
['adomani', 'github-actions'] |
nobody |
409-8943 1 year ago |
451-3852 1 year ago |
0-0 0 seconds |
13512 |
adomani author:adomani |
test: count all |
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict |
85/0 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter.lean,Mathlib/Tactic/Linter/Tally.lean |
4 |
0 |
[] |
nobody |
409-8943 1 year ago |
451-3725 1 year ago |
0-0 0 seconds |
12933 |
grunweg author:grunweg |
chore: replace some use of > or ≥ by < or ≤ |
These were flagged by the linter in #12879: it is easy to simple avoid > or ≥ in hypotheses or `have`s.
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict
awaiting-author
|
123/123 |
Archive/Imo/Imo1960Q1.lean,Archive/Imo/Imo1962Q1.lean,Archive/Imo/Imo1988Q6.lean,Archive/Imo/Imo2005Q3.lean,Archive/Imo/Imo2008Q2.lean,Archive/Imo/Imo2008Q4.lean,Archive/Imo/Imo2011Q5.lean,Archive/Imo/Imo2019Q4.lean,Archive/Wiedijk100Theorems/AreaOfACircle.lean,Archive/Wiedijk100Theorems/BallotProblem.lean,Mathlib/Algebra/DualNumber.lean,Mathlib/Algebra/Order/CauSeq/BigOperators.lean,Mathlib/Algebra/Order/Ring/Defs.lean,Mathlib/Algebra/Polynomial/Basic.lean,Mathlib/Algebra/Polynomial/Degree/Definitions.lean,Mathlib/Algebra/Star/CHSH.lean,Mathlib/Analysis/Analytic/Basic.lean,Mathlib/Analysis/Calculus/UniformLimitsDeriv.lean,Mathlib/Analysis/Complex/Hadamard.lean,Mathlib/Analysis/Complex/UpperHalfPlane/Basic.lean,Mathlib/Analysis/InnerProductSpace/Projection.lean,Mathlib/Analysis/Normed/Group/ControlledClosure.lean,Mathlib/Analysis/SpecialFunctions/Log/Base.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Basic.lean,Mathlib/Combinatorics/SimpleGraph/DegreeSum.lean,Mathlib/Combinatorics/SimpleGraph/LapMatrix.lean,Mathlib/Data/Complex/Basic.lean,Mathlib/Data/FP/Basic.lean,Mathlib/Data/Finset/Basic.lean,Mathlib/Data/Finsupp/Notation.lean,Mathlib/Data/Nat/Dist.lean,Mathlib/Data/Nat/Lattice.lean,Mathlib/Data/Nat/Parity.lean,Mathlib/Data/Ordmap/Ordset.lean,Mathlib/Data/PNat/Basic.lean,Mathlib/Data/UInt.lean,Mathlib/GroupTheory/Coxeter/Length.lean,Mathlib/MeasureTheory/Constructions/Polish.lean,Mathlib/MeasureTheory/Covering/Besicovitch.lean,Mathlib/MeasureTheory/Covering/Vitali.lean,Mathlib/MeasureTheory/Covering/VitaliFamily.lean,Mathlib/MeasureTheory/Integral/Layercake.lean,Mathlib/NumberTheory/LegendreSymbol/JacobiSymbol.lean,Mathlib/NumberTheory/Padics/Hensel.lean,Mathlib/NumberTheory/Padics/PadicNorm.lean,Mathlib/NumberTheory/PellMatiyasevic.lean,Mathlib/NumberTheory/Rayleigh.lean,Mathlib/Probability/Process/Stopping.lean,Mathlib/Tactic/CancelDenoms/Core.lean,Mathlib/Tactic/IntervalCases.lean,Mathlib/Tactic/Linarith/Lemmas.lean,Mathlib/Tactic/Linarith/Oracle/FourierMotzkin.lean,Mathlib/Tactic/NormNum/GCD.lean,Mathlib/Tactic/NormNum/Inv.lean,Mathlib/Tactic/Ring/Basic.lean,Mathlib/Topology/Category/Profinite/Nobeling.lean,Mathlib/Topology/ContinuousFunction/Bounded.lean,Mathlib/Topology/MetricSpace/CauSeqFilter.lean,Mathlib/Topology/Sequences.lean,test/LibrarySearch/basic.lean,test/Use.lean,test/cancel_denoms.lean,test/linarith.lean,test/norm_cast.lean |
64 |
6 |
['YaelDillies', 'github-actions', 'grunweg'] |
nobody |
409-8942 1 year ago |
422-18533 1 year ago |
0-55655 15 hours |
12416 |
adomani author:adomani |
chore: remove some cdots |
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict |
3830/3239 |
Archive/Imo/Imo1972Q5.lean,Archive/Imo/Imo2006Q5.lean,Archive/Imo/Imo2008Q2.lean,Archive/Imo/Imo2021Q1.lean,Archive/Wiedijk100Theorems/AbelRuffini.lean,Archive/Wiedijk100Theorems/BallotProblem.lean,Archive/Wiedijk100Theorems/BirthdayProblem.lean,Archive/Wiedijk100Theorems/BuffonsNeedle.lean,Archive/Wiedijk100Theorems/CubingACube.lean,Archive/Wiedijk100Theorems/FriendshipGraphs.lean,Archive/Wiedijk100Theorems/Partition.lean,Counterexamples/Cyclotomic105.lean,Counterexamples/DirectSumIsInternal.lean,Mathlib.lean,Mathlib/Algebra/Algebra/Spectrum.lean,Mathlib/Algebra/BigOperators/Finprod.lean,Mathlib/Algebra/BigOperators/List/Basic.lean,Mathlib/Algebra/Category/GroupCat/Colimits.lean,Mathlib/Algebra/Category/ModuleCat/Images.lean,Mathlib/Algebra/Category/Ring/Constructions.lean,Mathlib/Algebra/CharP/Quotient.lean,Mathlib/Algebra/ContinuedFractions/Computation/Approximations.lean,Mathlib/Algebra/DirectLimit.lean,Mathlib/Algebra/DirectSum/Internal.lean,Mathlib/Algebra/GCDMonoid/Finset.lean,Mathlib/Algebra/GeomSum.lean,Mathlib/Algebra/Group/UniqueProds.lean,Mathlib/Algebra/GroupPower/Order.lean,Mathlib/Algebra/GroupWithZero/WithZero.lean,Mathlib/Algebra/Homology/Exact.lean,Mathlib/Algebra/Homology/HomotopyCategory/HomComplex.lean,Mathlib/Algebra/Homology/HomotopyCategory/Triangulated.lean,Mathlib/Algebra/Homology/LocalCohomology.lean,Mathlib/Algebra/Homology/TotalComplex.lean,Mathlib/Algebra/Lie/DirectSum.lean,Mathlib/Algebra/Lie/IdealOperations.lean,Mathlib/Algebra/Lie/Nilpotent.lean,Mathlib/Algebra/Lie/Weights/Basic.lean,Mathlib/Algebra/Module/DedekindDomain.lean,Mathlib/Algebra/Module/LinearMap/End.lean,Mathlib/Algebra/Module/LocalizedModule.lean,Mathlib/Algebra/Module/PID.lean,Mathlib/Algebra/Module/Submodule/Bilinear.lean,Mathlib/Algebra/Module/Torsion.lean,Mathlib/Algebra/Module/Zlattice/Basic.lean,Mathlib/Algebra/MonoidAlgebra/Basic.lean,Mathlib/Algebra/MonoidAlgebra/Degree.lean,Mathlib/Algebra/MonoidAlgebra/Ideal.lean,Mathlib/Algebra/MvPolynomial/Variables.lean,Mathlib/Algebra/Order/Archimedean.lean,Mathlib/Algebra/Order/BigOperators/Group/List.lean,Mathlib/Algebra/Order/CauSeq/BigOperators.lean,Mathlib/Algebra/Order/CompleteField.lean,Mathlib/Algebra/Order/Field/Basic.lean,Mathlib/Algebra/Order/Group/Abs.lean,Mathlib/Algebra/Order/Group/Int.lean,Mathlib/Algebra/Order/Group/MinMax.lean,Mathlib/Algebra/Order/Interval/Basic.lean,Mathlib/Algebra/Order/Pointwise.lean,Mathlib/Algebra/Order/Sub/Defs.lean,Mathlib/Algebra/Polynomial/BigOperators.lean,Mathlib/Algebra/Polynomial/Degree/Definitions.lean,Mathlib/Algebra/Polynomial/Derivative.lean,Mathlib/Algebra/Polynomial/Div.lean,Mathlib/Algebra/Polynomial/FieldDivision.lean,Mathlib/Algebra/Polynomial/Module/Basic.lean,Mathlib/Algebra/Polynomial/PartialFractions.lean,Mathlib/Algebra/Polynomial/Reverse.lean,Mathlib/Algebra/Polynomial/RingDivision.lean,Mathlib/Algebra/Polynomial/UnitTrinomial.lean,Mathlib/Algebra/Quandle.lean,Mathlib/Algebra/Quaternion.lean,Mathlib/AlgebraicGeometry/AffineScheme.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Affine.lean,Mathlib/AlgebraicGeometry/FunctionField.lean,Mathlib/AlgebraicGeometry/Gluing.lean,Mathlib/AlgebraicGeometry/Morphisms/Basic.lean,Mathlib/AlgebraicGeometry/Morphisms/QuasiCompact.lean,Mathlib/AlgebraicGeometry/Morphisms/QuasiSeparated.lean,Mathlib/AlgebraicGeometry/Morphisms/RingHomProperties.lean,Mathlib/AlgebraicGeometry/OpenImmersion.lean,Mathlib/AlgebraicGeometry/ProjectiveSpectrum/Scheme.lean,Mathlib/AlgebraicGeometry/Properties.lean,Mathlib/AlgebraicGeometry/Pullbacks.lean,Mathlib/AlgebraicGeometry/StructureSheaf.lean,Mathlib/AlgebraicTopology/SimplexCategory.lean,Mathlib/AlgebraicTopology/SplitSimplicialObject.lean,Mathlib/Analysis/Analytic/Composition.lean,Mathlib/Analysis/Analytic/IsolatedZeros.lean,Mathlib/Analysis/BoundedVariation.lean,Mathlib/Analysis/BoxIntegral/Box/Basic.lean,Mathlib/Analysis/BoxIntegral/Partition/Basic.lean,Mathlib/Analysis/Calculus/ContDiff/Basic.lean,Mathlib/Analysis/Calculus/Deriv/Slope.lean,Mathlib/Analysis/Calculus/FDeriv/Basic.lean,Mathlib/Analysis/Calculus/FDeriv/Extend.lean,Mathlib/Analysis/Calculus/InverseFunctionTheorem/ApproximatesLinearOn.lean,Mathlib/Analysis/Calculus/LocalExtr/Basic.lean,Mathlib/Analysis/Calculus/ParametricIntegral.lean,Mathlib/Analysis/Calculus/TangentCone.lean |
608 |
0 |
[] |
nobody |
409-8942 1 year ago |
501-10940 1 year ago |
0-0 0 seconds |
12528 |
adomani author:adomani |
test: autotranslations Bot --> Top |
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict |
350/294 |
Mathlib.lean,Mathlib/Order/WithBot.lean,Mathlib/Tactic.lean,Mathlib/Tactic/MinMax.lean,test/MinMax.lean |
5 |
0 |
[] |
nobody |
409-8942 1 year ago |
479-9084 1 year ago |
0-0 0 seconds |
12473 |
adomani author:adomani |
first translations |
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict |
424/265 |
Mathlib.lean,Mathlib/Order/Lattice.lean,Mathlib/Order/WithBot.lean,Mathlib/Tactic.lean,Mathlib/Tactic/MinMax.lean |
5 |
0 |
[] |
nobody |
409-8942 1 year ago |
479-9085 1 year ago |
0-0 0 seconds |
12608 |
eric-wieser author:eric-wieser |
feat: allow `nsmul` / `zsmul` to be omitted again, with a warning |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-meta
merge-conflict
awaiting-author
label:t-algebra$ |
118/2 |
Mathlib.lean,Mathlib/Algebra/Group/Defs.lean,Mathlib/Tactic.lean,Mathlib/Tactic/DefaultFieldLinter.lean,scripts/noshake.json,test/default_field_linter.lean |
6 |
12 |
['YaelDillies', 'eric-wieser', 'fpvandoorn', 'github-actions'] |
nobody |
409-8942 1 year ago |
458-4006 1 year ago |
5-72414 5 days |
12637 |
adomani author:adomani |
translation: MonoidAlgebra to AddMonoidAlgebra |
[Zulip discussion](https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/merge.20Add-MonoidAlgebra)
* #12646 was found as a consequence of unification.
* #12659 the typo `single 1 1` for `single 0 1`.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-meta
merge-conflict
label:t-algebra$ |
615/986 |
Mathlib.lean,Mathlib/Algebra/MonoidAlgebra/Basic.lean,Mathlib/Algebra/MonoidAlgebra/Division.lean,Mathlib/Algebra/MvPolynomial/Basic.lean,Mathlib/Tactic.lean,Mathlib/Tactic/MinMaxTwo.lean,scripts/noshake.json |
7 |
0 |
[] |
nobody |
409-8942 1 year ago |
430-76042 1 year ago |
0-0 0 seconds |
12679 |
MichaelStollBayreuth author:MichaelStollBayreuth |
perf(NumberTheory/RamificationInertia): speed up slow file |
A repetition of the earlier experiment at [#12412](https://github.com/leanprover-community/mathlib4/pull/12412) with Lean 4.8.0-rc1.
This time, I tried not to introduce local instances if possible, but instead to tweak instance priorities.
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict
WIP
|
57/14 |
Mathlib/NumberTheory/RamificationInertia.lean |
1 |
3 |
['MichaelStollBayreuth', 'github-actions', 'leanprover-bot'] |
nobody |
409-8942 1 year ago |
466-54487 1 year ago |
0-0 0 seconds |
12588 |
adomani author:adomani |
remove trailingDegree |
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict |
1280/979 |
Mathlib.lean,Mathlib/Algebra/MonoidAlgebra/Basic.lean,Mathlib/Algebra/Polynomial/Degree/Definitions.lean,Mathlib/Algebra/Polynomial/Degree/TrailingDegree.lean,Mathlib/Algebra/Polynomial/Div.lean,Mathlib/Algebra/Polynomial/Mirror.lean,Mathlib/Order/WithBot.lean,Mathlib/Tactic.lean,Mathlib/Tactic/MinMax.lean,Mathlib/Tactic/MinMaxTwo.lean,test/MinMax.lean |
11 |
0 |
[] |
nobody |
409-8942 1 year ago |
497-12518 1 year ago |
0-0 0 seconds |
12936 |
mattrobball author:mattrobball |
chore(Quiver.Opposite): make `Quiver.Hom.op/unop` `abbrev`'s |
These are wrappers around the constructor and projection for `Opposite Quiver.Hom _ _`. The projection itself is reducible and with structure eta built in to defeq it seems like we might be making Lean work harder than is necessary.
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict |
39/34 |
Mathlib/Algebra/Homology/ShortComplex/Homology.lean,Mathlib/Algebra/Homology/ShortComplex/RightHomology.lean,Mathlib/CategoryTheory/Idempotents/Basic.lean,Mathlib/CategoryTheory/Limits/HasLimits.lean,Mathlib/CategoryTheory/Limits/Opposites.lean,Mathlib/CategoryTheory/Opposites.lean,Mathlib/CategoryTheory/Sites/CoverLifting.lean,Mathlib/CategoryTheory/Subobject/Comma.lean,Mathlib/CategoryTheory/Triangulated/Opposite.lean,Mathlib/Combinatorics/Quiver/Basic.lean |
10 |
9 |
['YaelDillies', 'kim-em', 'leanprover-bot', 'mattrobball'] |
nobody |
409-8942 1 year ago |
476-61334 1 year ago |
0-0 0 seconds |
12934 |
grunweg author:grunweg |
chore: replace more uses of > or ≥ by < or ≤ |
These were flagged by the linter in https://github.com/leanprover-community/mathlib4/pull/12879: it is easy to simple avoid > or ≥ in hypotheses or haves.
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict
awaiting-author
help-wanted
|
41/42 |
Archive/Imo/Imo1962Q1.lean,Archive/Imo/Imo1988Q6.lean,Archive/Imo/Imo1994Q1.lean,Archive/Imo/Imo2005Q3.lean,Archive/Imo/Imo2006Q3.lean,Archive/Imo/Imo2008Q2.lean,Archive/Imo/Imo2008Q3.lean,Archive/Imo/Imo2019Q4.lean,Archive/Sensitivity.lean,Archive/Wiedijk100Theorems/CubingACube.lean,Mathlib/Tactic/Linarith/Datatypes.lean,test/cancel_denoms.lean,test/congr.lean,test/interval_cases.lean,test/observe.lean |
15 |
11 |
['YaelDillies', 'adomani', 'github-actions', 'grunweg', 'jcommelin', 'urkud'] |
nobody |
409-8942 1 year ago |
422-18539 1 year ago |
1-73101 1 day |
12465 |
rosborn author:rosborn |
style: Change Subtype.val to (↑) |
---
This is a test to see replacing `Subtype.val` with `(↑)` where appropriate.
After performing the rewrite, some of the types subtly changed in a difficult to detect manner.
Before the change, `openEmbedding' _` had type `OpenEmbedding Subtype.val` where `Subtype.val` expanded as `@Subtype.val α fun x ↦ x ∈ U : ↥U → α`. After the change, `Subtype.val` expands to `@Subtype.val α fun x ↦ x ∈ ↑U : { x // x ∈ ↑U } → α`. This caused some later proofs to fail due to the different definition.
In a similar case, within the proof of `mfderiv_coe_sphere_injective` on line 553 `Subtype.val` expanded as `@Subtype.val E fun x ↦ x ∈ (Submodule.span ℝ {↑(-v)})ᗮ : ↥(Submodule.span ℝ {↑(-v)})ᗮ → E`.
After changing to `(↑)`, it expanded to `@Subtype.val E fun x ↦ x ∈ ↑(Submodule.span ℝ {↑(-v)})ᗮ : { x // x ∈ ↑(Submodule.span ℝ {↑(-v)})ᗮ } → E`. One benefit to using `(↑)` was that it lead to a shorter proof as `ContinuousLinearEquiv.coe_coe` could be removed on line 559.
In general, this subtle change in types is basically impossible to detect without a tool like leaff.
[](https://gitpod.io/from-referrer/)
|
merge-conflict |
50/50 |
Mathlib/Analysis/InnerProductSpace/Basic.lean,Mathlib/Analysis/Normed/Group/Hom.lean,Mathlib/CategoryTheory/Generator.lean,Mathlib/CategoryTheory/Limits/Shapes/Types.lean,Mathlib/CategoryTheory/Subobject/Types.lean,Mathlib/Data/Fin/Basic.lean,Mathlib/Data/Set/Function.lean,Mathlib/Data/Set/Image.lean,Mathlib/Data/Setoid/Basic.lean,Mathlib/Geometry/Manifold/ContMDiff/Basic.lean,Mathlib/Geometry/Manifold/Instances/Sphere.lean,Mathlib/Geometry/Manifold/LocalInvariantProperties.lean,Mathlib/GroupTheory/Subsemigroup/Operations.lean,Mathlib/LinearAlgebra/LinearIndependent.lean,Mathlib/Order/Directed.lean,Mathlib/Order/RelIso/Basic.lean,Mathlib/Order/RelIso/Set.lean,Mathlib/RingTheory/Artinian.lean,Mathlib/SetTheory/Cardinal/Cofinality.lean,Mathlib/SetTheory/Game/Basic.lean,Mathlib/SetTheory/Game/PGame.lean,Mathlib/SetTheory/Surreal/Basic.lean,Mathlib/Topology/Bornology/Constructions.lean,Mathlib/Topology/EMetricSpace/Lipschitz.lean,Mathlib/Topology/Germ.lean,Mathlib/Topology/UniformSpace/Basic.lean,Mathlib/Topology/UniformSpace/UniformConvergenceTopology.lean,Mathlib/Topology/UniformSpace/UniformEmbedding.lean |
28 |
1 |
['eric-wieser', 'rosborn'] |
nobody |
409-8942 1 year ago |
497-71133 1 year ago |
0-0 0 seconds |
11617 |
urkud author:urkud |
refactor(Finset): redefine Finset.diag, review API |
Redefine `Finset.diag` using `Finset.map`.
The new definition doesn't rely on `DecidableEq` and is much more computationally efficient.
Also review API and golf proofs here and there.
---
[](https://gitpod.io/from-referrer/)
|
t-logic
merge-conflict
awaiting-author
|
187/181 |
Archive/Imo/Imo1998Q2.lean,Mathlib.lean,Mathlib/Algebra/BigOperators/Basic.lean,Mathlib/Combinatorics/SimpleGraph/Regularity/Energy.lean,Mathlib/Combinatorics/SimpleGraph/Regularity/Increment.lean,Mathlib/Combinatorics/SimpleGraph/Regularity/Uniform.lean,Mathlib/Data/Finset/Diag.lean,Mathlib/Data/Finset/Image.lean,Mathlib/Data/Finset/Prod.lean,Mathlib/Data/Set/Image.lean,Mathlib/Data/Set/Prod.lean,Mathlib/Data/Sym/Card.lean,Mathlib/Data/Sym/Sym2.lean |
13 |
7 |
['YaelDillies', 'eric-wieser', 'urkud'] |
nobody |
409-8941 1 year ago |
531-47071 1 year ago |
1-12270 1 day |
12192 |
Ruben-VandeVelde author:Ruben-VandeVelde |
feat: generalize isLittleO_const_id_atTop/atBot |
From PNT+.
---
[](https://gitpod.io/from-referrer/)
|
t-analysis
merge-conflict
awaiting-author
|
10/4 |
Mathlib/Analysis/Asymptotics/Asymptotics.lean |
1 |
6 |
['Ruben-VandeVelde', 'llllvvuu', 'urkud'] |
nobody |
409-8941 1 year ago |
420-73208 1 year ago |
1-21749 1 day |
10444 |
urkud author:urkud |
doc(IsROrC): expand the docstring |
---
[](https://gitpod.io/from-referrer/) |
t-analysis
merge-conflict
awaiting-author
documentation
|
34/0 |
Mathlib/Data/IsROrC/Basic.lean |
1 |
9 |
['eric-wieser', 'kbuzzard', 'urkud'] |
nobody |
409-8940 1 year ago |
533-81232 1 year ago |
1-62352 1 day |
10024 |
ADedecker author:ADedecker |
feat: rename `connectedComponentOfOne` to `identityComponent`, prove that it is normal and open |
---
[](https://gitpod.io/from-referrer/)
|
t-topology
awaiting-CI
merge-conflict
|
58/24 |
Mathlib/FieldTheory/AbsoluteGaloisGroup.lean,Mathlib/Topology/Algebra/Group/Basic.lean,Mathlib/Topology/Algebra/Group/TopologicalAbelianization.lean,Mathlib/Topology/Algebra/OpenSubgroup.lean,Mathlib/Topology/Connected/Basic.lean |
5 |
0 |
[] |
nobody |
409-8940 1 year ago |
420-73797 1 year ago |
0-832 13 minutes |
10521 |
eric-wieser author:eric-wieser |
chore: generalize `IsBoundedLinearMap` to modules |
Most of the lemmas don't actually need the normed on the scalars at all.
---
[](https://gitpod.io/from-referrer/)
|
t-analysis
merge-conflict
awaiting-author
|
58/42 |
Mathlib/Analysis/NormedSpace/BoundedLinearMaps.lean |
1 |
3 |
['github-actions', 'j-loreaux', 'urkud'] |
nobody |
409-8940 1 year ago |
516-23002 1 year ago |
1-29105 1 day |
11100 |
eric-wieser author:eric-wieser |
feat(CategoryTheory/Limits): add `Functor.mapBinaryBiconeInv` |
---
- [ ] depends on: #11130
[](https://gitpod.io/from-referrer/)
It's tempting to try to prove something like
```lean
theorem Functor.mapBinaryBiconeInv_toCone [Limits.HasZeroMorphisms C]
[Limits.HasZeroMorphisms D]
(e : D ⥤ C) [IsEquivalence e] {X Y : D} (b : BinaryBicone (e.obj X) (e.obj Y)) :
(e.mapBinaryBiconeInv b).toCone =
(e.mapConeInv <| (Cones.postcompose (pairComp X Y e).symm.hom).obj b.toCone) := by
simp
sorry
theorem Functor.mapBinaryBiconeInv_toCocone [Limits.HasZeroMorphisms C]
[Limits.HasZeroMorphisms D]
(e : D ⥤ C) [IsEquivalence e] {X Y : D} (b : BinaryBicone (e.obj X) (e.obj Y)) :
(e.mapBinaryBiconeInv b).toCocone =
(e.mapCoconeInv <| (Cocones.precompose (pairComp X Y e).hom).obj b.toCocone) := by
sorry
```
but maybe equality is evil here |
t-category-theory
awaiting-CI
merge-conflict
|
52/0 |
Mathlib/CategoryTheory/Adjunction/Basic.lean,Mathlib/CategoryTheory/Equivalence.lean,Mathlib/CategoryTheory/Limits/Preserves/Shapes/Biproducts.lean |
3 |
6 |
['TwoFX', 'eric-wieser', 'leanprover-community-mathlib4-bot'] |
nobody |
409-8940 1 year ago |
430-76042 1 year ago |
0-0 0 seconds |
10721 |
urkud author:urkud |
feat(Order/FunLike): define `PointwiseLE` |
- introduce a mixin class `DFunLike.PointwiseLE`, use it to define `DFunLike.instPartialOrder`;
- add a generic `DFunLike.orderEmbeddingCoe`
- add `DFunLike.PointwiseLE` instances here and there.
With this refactor and #13022, I'm going to generalize lemmas like `MeasureTheory.ae_mono` to `OuterMeasureClass`.
---
- [x] depends on: #12983
[](https://gitpod.io/from-referrer/) |
t-logic
t-order
merge-conflict
|
123/50 |
Mathlib.lean,Mathlib/Algebra/Order/Hom/Ring.lean,Mathlib/Data/DFinsupp/Order.lean,Mathlib/Data/Finsupp/Order.lean,Mathlib/Data/FunLike/Basic.lean,Mathlib/Dynamics/Circle/RotationNumber/TranslationNumber.lean,Mathlib/GroupTheory/Congruence.lean,Mathlib/Order/FunLike.lean,Mathlib/Order/Heyting/Hom.lean,Mathlib/Order/Hom/Basic.lean,Mathlib/Order/Hom/Bounded.lean,Mathlib/Order/Hom/CompleteLattice.lean,Mathlib/Topology/Order/Hom/Basic.lean |
13 |
48 |
['YaelDillies', 'dupuisf', 'leanprover-community-mathlib4-bot', 'urkud'] |
nobody |
409-8940 1 year ago |
430-76042 1 year ago |
64-12826 64 days |
10594 |
lecopivo author:lecopivo |
feat: `fun_trans` function transformation tactic e.g. for computing derivatives |
feat: `fun_trans` function transformation tactic e.g. for computing derivatives
Function transformation tactic/simproc. For example it can be used for computing derivatives.
---
[](https://gitpod.io/from-referrer/)
|
t-meta
merge-conflict
WIP
|
1819/56 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/FunProp/Core.lean,Mathlib/Tactic/FunProp/Decl.lean,Mathlib/Tactic/FunProp/Elab.lean,Mathlib/Tactic/FunProp/FunctionData.lean,Mathlib/Tactic/FunProp/MorExt.lean,Mathlib/Tactic/FunProp/Theorems.lean,Mathlib/Tactic/FunTrans/Attr.lean,Mathlib/Tactic/FunTrans/Core.lean,Mathlib/Tactic/FunTrans/Decl.lean,Mathlib/Tactic/FunTrans/Elab.lean,Mathlib/Tactic/FunTrans/Theorems.lean,Mathlib/Tactic/FunTrans/Types.lean,test/fun_prop2.lean,test/fun_prop_dev.lean,test/fun_trans_dev.lean |
17 |
11 |
['github-actions'] |
nobody |
409-8940 1 year ago |
470-32599 1 year ago |
0-0 0 seconds |
10845 |
Shamrock-Frost author:Shamrock-Frost |
Refactor: Make MonoidalFunctor carry the data of an inverse |
We change the definition of a strong monoidal functor from a lax monoidal functor for which the unitor and tensorator are `IsIso` to a lax monoidal functor with the data of inverses for the unitor and tensorator. This requires fixing a lot of knock on effects.
---
This is a **draft PR**. I would like to talk with people on zulip before merging it, and plan ahead to when we have oplax/colax monoidal functors as well. I'm not sure the approach I took here where `MonoidalFunctor` inherits from `LaxMonoidalFunctor` is a good choice if we want to be lax/oplax symmetric.
[](https://gitpod.io/from-referrer/)
|
t-category-theory
RFC
merge-conflict
WIP
|
3799/1589 |
Mathlib/Algebra/Category/ModuleCat/Adjunctions.lean,Mathlib/Algebra/Homology/HomotopyCategory/DegreewiseSplit.lean,Mathlib/CategoryTheory/Adjunction/Basic.lean,Mathlib/CategoryTheory/Adjunction/Mates.lean,Mathlib/CategoryTheory/Adjunction/Opposites.lean,Mathlib/CategoryTheory/Adjunction/Prod.lean,Mathlib/CategoryTheory/Adjunction/Whiskering.lean,Mathlib/CategoryTheory/Bicategory/End.lean,Mathlib/CategoryTheory/Bicategory/SingleObj.lean,Mathlib/CategoryTheory/CatCommSq.lean,Mathlib/CategoryTheory/CatSquares.lean,Mathlib/CategoryTheory/Enriched/Basic.lean,Mathlib/CategoryTheory/Equivalence.lean,Mathlib/CategoryTheory/Iso.lean,Mathlib/CategoryTheory/Monoidal/Adjunction.lean,Mathlib/CategoryTheory/Monoidal/Braided.lean,Mathlib/CategoryTheory/Monoidal/Category.lean,Mathlib/CategoryTheory/Monoidal/Center.lean,Mathlib/CategoryTheory/Monoidal/CommMon_.lean,Mathlib/CategoryTheory/Monoidal/Discrete.lean,Mathlib/CategoryTheory/Monoidal/End.lean,Mathlib/CategoryTheory/Monoidal/Free/Basic.lean,Mathlib/CategoryTheory/Monoidal/Functor.lean,Mathlib/CategoryTheory/Monoidal/Limits.lean,Mathlib/CategoryTheory/Monoidal/Mon_.lean,Mathlib/CategoryTheory/Monoidal/NaturalTransformation.lean,Mathlib/CategoryTheory/Monoidal/Opposite.lean,Mathlib/CategoryTheory/Monoidal/Rigid/FunctorCategory.lean,Mathlib/CategoryTheory/Monoidal/Rigid/OfEquivalence.lean,Mathlib/CategoryTheory/Monoidal/Subcategory.lean,Mathlib/CategoryTheory/Monoidal/Transport.lean,Mathlib/CategoryTheory/Monoidal/Types/Basic.lean,Mathlib/CategoryTheory/Opposites.lean,Mathlib/CategoryTheory/Products/Associator.lean,Mathlib/CategoryTheory/Products/Basic.lean,Mathlib/CategoryTheory/Shift/Basic.lean,Mathlib/CategoryTheory/Shift/Pullback.lean,Mathlib/CategoryTheory/Whiskering.lean,Mathlib/RepresentationTheory/Action/Monoidal.lean,Mathlib/RepresentationTheory/GroupCohomology/Resolution.lean,Mathlib/RepresentationTheory/Rep.lean |
41 |
7 |
['Shamrock-Frost', 'joelriou'] |
nobody |
409-8940 1 year ago |
564-33473 1 year ago |
0-0 0 seconds |
9564 |
AntoineChambert-Loir author:AntoineChambert-Loir |
weaken commutativity assumptions for AdjoinRoot.lift and AdjoinRoot.liftHom |
I weaken a commutativity assumption for docs#AdjoinRoot.liftHom that the target algebra be commutative. It is only assumed to be a Semiring.
For that, I need to generalize docs#AdjoinRoot.lift which takes `i : R ->+* S`, `a : S` with `f.eval₂ i a = 0` and defines `AdjoinRoot f ->+* S` that extends `i ` and sends `AdjoinRoot.root f` to `a`.
---
The initial version of the PR was to define `AdjoinRoot.lift'` where `S` is only a Semiring, with the additional assumption `hcomm : ∀ r, Commute (i r) a` that the element `a` commutes with the image of `i`.
@jcommelin suggested to provide this argument as an `autoParam`, filled in by an ad hoc `commutativity` tactic. However, such an argument cannot be made implicit and a first version required to have this argument given each time, most of the time by `_`, even for all subsequent lemmas, `AdjoinRoot.lift_mk`, etc.
To avoid this, I tried to make this assumption a `⦃hcomm : ∀ r, Commute (i r) a⦄`. This appears to have some side effects that proofs using an `exact` tactic or in term mode do not work well, but one can resort on `by simp […]`. Maybe @eric-wieser or @Vierkantor will have opinions on that. In some cases one can still give the argument as `(hcomm := by commutativity)`.
(There are 3 options :
- separate lemmas for the fully commutative case and for the case where a proof is needed
- using the `commutativity` tactic, but with an argument `_` sometimes
- using the optional argument.)
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
WIP
label:t-algebra$ |
146/30 |
Mathlib.lean,Mathlib/Algebra/Algebra/Basic.lean,Mathlib/Algebra/Algebra/Hom.lean,Mathlib/Algebra/Group/Commute/Defs.lean,Mathlib/RingTheory/AdjoinRoot.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Commutativity.lean,Mathlib/Tactic/Commutativity/Init.lean |
8 |
14 |
['AntoineChambert-Loir', 'Vierkantor', 'eric-wieser', 'jcommelin'] |
nobody |
409-8939 1 year ago |
430-76042 1 year ago |
16-24540 16 days |
9504 |
alreadydone author:alreadydone |
chore: remove some IsSeparable assumptions |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
WIP
label:t-algebra$ |
41/14 |
Mathlib/NumberTheory/NumberField/Norm.lean,Mathlib/RingTheory/Norm.lean |
2 |
0 |
[] |
nobody |
409-8939 1 year ago |
497-70123 1 year ago |
0-0 0 seconds |
9487 |
eric-wieser author:eric-wieser |
feat: the exponential of dual numbers over non-commutative rings |
This is a work in progress, as I don't know my way around the measure theory library.
---
- [x] depends on: #9489
- [x] depends on: #9486
- [x] depends on: #10427
- [ ] depends on: #10452
[](https://gitpod.io/from-referrer/)
|
t-measure-probability
t-algebra
t-analysis
merge-conflict
WIP
label:t-algebra$ |
97/0 |
Mathlib/Analysis/NormedSpace/TrivSqZeroExt.lean |
1 |
7 |
['github-actions', 'leanprover-community-mathlib4-bot'] |
nobody |
409-8939 1 year ago |
414-4008 1 year ago |
0-0 0 seconds |
8616 |
eric-wieser author:eric-wieser |
feat(Algebra/FreeAlgebra): add right action and `IsCentralScalar` |
---
- [ ] depends on: #8652
[](https://gitpod.io/from-referrer/)
|
t-algebra
awaiting-CI
merge-conflict
label:t-algebra$ |
30/8 |
Mathlib/Algebra/FreeAlgebra.lean |
1 |
1 |
['leanprover-community-mathlib4-bot'] |
nobody |
409-8939 1 year ago |
430-76042 1 year ago |
0-0 0 seconds |
8582 |
eric-wieser author:eric-wieser |
wip |
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict |
3/7 |
Mathlib/Algebra/Category/AlgebraCat/Monoidal.lean,Mathlib/LinearAlgebra/TensorProduct.lean |
2 |
4 |
['eric-wieser', 'leanprover-bot'] |
nobody |
409-8939 1 year ago |
659-82195 1 year ago |
0-0 0 seconds |
8503 |
thorimur author:thorimur |
feat: meta utils for `refine?` |
This PR introduces some metaprogramming infrastructure and utilities that are necessary for `refine?` (#8364).
* `elabTermWithHoles'` (and `withCollectingNewGoalsFrom'`): a more configurable version of `elabTermWithHoles`, which allows: preserving the initial mvar type; *not* tagging untagged goals; and postponing mvars.
* Some `Syntax` and `TSyntax` functionality, including:
* `TSyntax.map`(`M`), for acting on `TSyntax` with functions `f : Syntax -> (m) Syntax`
* Range operations: `includes` and `isEqByRange`
* `setTrailingInfoBy?` and `unsetOriginalTrailing`, which is like `unsetTrailing`, but behaves as expected.
* `Term.withoutModifyingState`, which does not allow unknown mvarIds to escape via the infotree
* `hasNewErrors`, which runs a monad computation and returns the value along with `true` or `false` depending on whether new error messages have been logged
* the option `pp.anonymousMVarSuffixes`, which can be set to `false` to replace all numeric suffixes of anonymous mvars with `✝`, which is useful in tandem with `#guard_msgs` for tests (but is essentially a workaround—although it can make some tactic states more legible).
---
I'm open to suggestions on the location and name of the option/delaborator used for trimming the numeric suffixes of anonymous mvar names (which is used in the tests)—including whether or not it should exist in the first place, as it's essentially just a workaround.
[](https://gitpod.io/from-referrer/)
|
t-meta
merge-conflict
awaiting-author
|
312/5 |
Mathlib.lean,Mathlib/Lean/CoreM.lean,Mathlib/Lean/Elab/Tactic/ElabTerm.lean,Mathlib/Lean/Elab/Term.lean,Mathlib/Util/Delaborators.lean,Mathlib/Util/Syntax.lean |
6 |
2 |
['kmill', 'thorimur'] |
kmill assignee:kmill |
409-8939 1 year ago |
611-19237 1 year ago |
38-46649 38 days |
9252 |
FR-vdash-bot author:FR-vdash-bot |
chore: remove redundant covariance instances, add priority |
I noticed that the following code is surprisingly slow.
``` lean
import Mathlib
count_heartbeats in
example {n : ℕ} : CovariantClass (Fin (n + 1)) (Fin (n + 1)) (· + ·) (· < ·) := by
try infer_instance
sorry
```
This PR removed some redundant instances. The heartbeats have dropped from 19118 to 11450 (still too slow).
Lean4 still seems to make some redundant attempts. See also https://github.com/leanprover-community/mathlib4/issues/6646#issuecomment-1691792488.
---
[](https://gitpod.io/from-referrer/)
|
slow-typeclass-synthesis
t-order
t-algebra
merge-conflict
awaiting-author
WIP
label:t-algebra$ |
40/32 |
Mathlib/Algebra/CovariantAndContravariant.lean,Mathlib/Algebra/Order/Group/Defs.lean,Mathlib/Algebra/Order/Monoid/Defs.lean,Mathlib/CategoryTheory/Abelian/DiagramLemmas/Four.lean |
4 |
8 |
['FR-vdash-bot', 'leanprover-bot', 'urkud'] |
nobody |
409-8939 1 year ago |
467-52364 1 year ago |
0-0 0 seconds |
8788 |
FMLJohn author:FMLJohn |
feat(Algebra/Module/GradeZeroModule): if `A` is a graded semiring and `M` is a graded `A`-module, then each grade of `M` is a module over the 0-th grade of `A`. |
---
- [ ] depends on: #8187
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
label:t-algebra$ |
237/4 |
Mathlib.lean,Mathlib/Algebra/DirectSum/Internal.lean,Mathlib/Algebra/GradedMonoid.lean,Mathlib/Algebra/Module/GradeZeroModule.lean,Mathlib/RingTheory/GradedAlgebra/Basic.lean,Mathlib/RingTheory/GradedAlgebra/Noetherian.lean |
6 |
4 |
['FMLJohn', 'github-actions', 'leanprover-community-mathlib4-bot'] |
nobody |
409-8939 1 year ago |
442-83241 1 year ago |
0-0 0 seconds |
9570 |
eric-wieser author:eric-wieser |
feat(Algebra/Star): Non-commutative generalization of `StarModule` |
[Zulip thread](https://leanprover.zulipchat.com/#narrow/stream/116395-maths/topic/Star.20modules.20over.20non-commutative.20scalars/near/383664005).
Until we address #7152, we have to have both `StarModule` and `StarModule'`.
To prove this generalization is useful, this shows that with it as an assumption, `TrivSqZeroExt` is a `StarRing`.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
awaiting-CI
merge-conflict
WIP
label:t-algebra$ |
66/6 |
Mathlib/Algebra/Star/Basic.lean,Mathlib/Algebra/Star/Pi.lean,Mathlib/Algebra/Star/Prod.lean,Mathlib/Algebra/TrivSqZeroExt.lean |
4 |
0 |
[] |
nobody |
409-8939 1 year ago |
501-85545 1 year ago |
0-0 0 seconds |
8906 |
jjaassoonn author:jjaassoonn |
feat: add some missing lemmas about linear algebra |
---
- [ ] depends on: #8905 [lifting injective modules to higher universe]
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
awaiting-author
label:t-algebra$ |
45/1 |
Mathlib/Algebra/Category/ModuleCat/Basic.lean,Mathlib/Algebra/Module/Injective.lean,Mathlib/LinearAlgebra/Basic.lean,Mathlib/LinearAlgebra/BilinearMap.lean |
4 |
21 |
['AntoineChambert-Loir', 'alreadydone', 'jjaassoonn', 'leanprover-community-mathlib4-bot'] |
nobody |
409-8939 1 year ago |
510-45068 1 year ago |
0-0 0 seconds |
8658 |
eric-wieser author:eric-wieser |
feat: support right actions for `Con` |
This adds a new `Con.CompatibleSMul` typeclass that captures exactly the condition when `smul` descends to the quotient.
I was not quite able to merge this with `MulAction.QuotientAction`:
* The imports are such that the congruence relation `QuotientGroup.con` is not yet available in that file
* `QuotientGroup.con` requires the subgroup to be normal, while `MulAction.QuotientAction` does not
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
awaiting-author
label:t-algebra$ |
80/18 |
Mathlib/GroupTheory/Congruence.lean,Mathlib/RingTheory/Congruence.lean |
2 |
6 |
['YaelDillies', 'eric-wieser'] |
nobody |
409-8939 1 year ago |
458-73993 1 year ago |
29-65537 29 days |
9642 |
eric-wieser author:eric-wieser |
refactor(Analysis/Normed/{Group/Field}/Basic): Let `extends` generate the repeated fields |
New-style structure shenanigans mean that instance constructors randomly complain about a missing field that can be found with `__ : MetricSpace _ := infer_instance`.
---
[](https://gitpod.io/from-referrer/)
I will write a longer PR description for this once CI is happy
|
t-analysis
merge-conflict
awaiting-author
WIP
help-wanted
|
122/202 |
Mathlib/Analysis/Calculus/ContDiff/Basic.lean,Mathlib/Analysis/Complex/Basic.lean,Mathlib/Analysis/Matrix.lean,Mathlib/Analysis/Normed/Field/Basic.lean,Mathlib/Analysis/Normed/Group/Basic.lean,Mathlib/Analysis/Normed/Group/Completion.lean,Mathlib/Analysis/Normed/Order/Basic.lean,Mathlib/Analysis/NormedSpace/ProdLp.lean,Mathlib/Analysis/NormedSpace/Star/Matrix.lean,Mathlib/Analysis/NormedSpace/Unitization.lean,Mathlib/Analysis/Quaternion.lean,Mathlib/Geometry/Manifold/Instances/Sphere.lean,Mathlib/InformationTheory/Hamming.lean,Mathlib/MeasureTheory/Measure/Lebesgue/VolumeOfBalls.lean,Mathlib/NumberTheory/NumberField/CanonicalEmbedding.lean,Mathlib/NumberTheory/Padics/PadicIntegers.lean,Mathlib/Topology/ContinuousFunction/Bounded.lean |
17 |
11 |
['eric-wieser', 'leanprover-bot', 'urkud'] |
nobody |
409-8939 1 year ago |
586-75241 1 year ago |
0-0 0 seconds |
8519 |
eric-wieser author:eric-wieser |
refactor(LinearAlgebra/TensorProduct): golf using `liftAddHom` |
This new `TensorProduct.liftAddHom` doesn't require bilinearity, only that scalar multiplication can be moved between the arguments.
While in theory we only need the `AddMonoidHom` version as it offers exactly the same generality, we first provide an unbundled `liftFun` as this seems to give a sizeable performance boost if used in downstream `lift` variants.
---
- [x] depends on: #8571
- [x] depends on: #8584
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
awaiting-author
label:t-algebra$ |
53/50 |
Mathlib/Algebra/Category/AlgebraCat/Monoidal.lean,Mathlib/LinearAlgebra/TensorProduct.lean,Mathlib/LinearAlgebra/TensorProduct/Tower.lean |
3 |
28 |
['bustercopley', 'eric-wieser', 'jcommelin', 'jjaassoonn', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'mathlib-bors'] |
nobody |
409-8939 1 year ago |
557-67654 1 year ago |
5-6524 5 days |
9146 |
laughinggas author:laughinggas |
feat(Data/ZMod/Defs): Topological structure on `ZMod` |
Added a discrete topology structure to `ZMod n` for all `n`
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-topology
merge-conflict
awaiting-author
label:t-algebra$ |
55/3 |
Mathlib.lean,Mathlib/Topology/Algebra/Constructions.lean,Mathlib/Topology/Algebra/Group/Basic.lean,Mathlib/Topology/Instances/ZMod.lean,Mathlib/Topology/Maps.lean |
5 |
61 |
['YaelDillies', 'eric-wieser', 'github-actions', 'jcommelin', 'laughinggas', 'mo271', 'urkud'] |
nobody |
409-8939 1 year ago |
590-17067 1 year ago |
7-6153 7 days |
8585 |
thorimur author:thorimur |
chore: bench lean4#2944 |
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict |
1/1 |
lean-toolchain |
1 |
2 |
['leanprover-bot', 'thorimur'] |
nobody |
409-8939 1 year ago |
660-14117 1 year ago* |
0-0 0 seconds* |
9356 |
alexjbest author:alexjbest |
feat: assumption? |
A little helper for replacing `assumption`s with `exact` statements quickly
---
If this is approved I will add tests
This begs the question of whether it might simply be better to add some sort of code action for "replace with trythis output"
[](https://gitpod.io/from-referrer/)
|
t-meta
merge-conflict
awaiting-author
|
24/0 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Common.lean,Mathlib/Tactic/TryAssumption.lean |
4 |
5 |
['alexjbest', 'j-loreaux', 'jcommelin'] |
nobody |
409-8939 1 year ago |
592-29336 1 year ago |
19-26304 19 days |
9229 |
eric-wieser author:eric-wieser |
refactor(Algebra/GradedMonoid): Use `HMul` to define `GMul` |
This make the notation much nicer, but I'm pretty sure this is a bad idea for performance / ambiguity reasons.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
WIP
label:t-algebra$ |
114/125 |
Mathlib/Algebra/DirectSum/Algebra.lean,Mathlib/Algebra/DirectSum/Internal.lean,Mathlib/Algebra/DirectSum/Ring.lean,Mathlib/Algebra/GradedMonoid.lean,Mathlib/Algebra/GradedMulAction.lean,Mathlib/Algebra/Module/GradedModule.lean,Mathlib/Algebra/MonoidAlgebra/ToDirectSum.lean,Mathlib/LinearAlgebra/TensorAlgebra/ToTensorPower.lean,Mathlib/LinearAlgebra/TensorPower.lean,Mathlib/LinearAlgebra/TensorProduct/Graded/Internal.lean,Mathlib/RingTheory/GradedAlgebra/Basic.lean |
11 |
6 |
['eric-wieser', 'leanprover-bot'] |
nobody |
409-8939 1 year ago |
572-85056 1 year ago |
0-0 0 seconds |
8961 |
eric-wieser author:eric-wieser |
refactor: use the coinduced topology on ULift |
---
- [x] depends on: #8958
[](https://gitpod.io/from-referrer/)
|
awaiting-CI
merge-conflict
please-adopt
awaiting-author
|
46/14 |
Mathlib/Analysis/Normed/Group/Basic.lean,Mathlib/Topology/Bornology/Constructions.lean,Mathlib/Topology/Constructions.lean |
3 |
6 |
['eric-wieser', 'github-actions', 'leanprover-community-mathlib4-bot', 'urkud'] |
nobody |
409-8939 1 year ago |
597-1183 1 year ago |
0-0 0 seconds |
9354 |
chenyili0818 author:chenyili0818 |
feat: monotonicity of gradient on convex real-valued functions |
This file is based on Mathlib.Analysis.Calculus.Gradient.Basic, and describes the calculation properties
co-authored-by: Ziyu Wang [tropicalfish910@gmail.com](mailto:tropicalfish910@gmail.com)
---
[](https://gitpod.io/from-referrer/)
|
t-analysis
merge-conflict
awaiting-author
|
540/0 |
Mathlib.lean,Mathlib/Analysis/Convex/ConvexFunction.lean |
2 |
15 |
['github-actions', 'winstonyin'] |
nobody |
409-8939 1 year ago |
539-62028 1 year ago |
22-72922 22 days |
9482 |
yuma-mizuno author:yuma-mizuno |
refactor(CategoryTheory/Monoidal): add `LaxMonoidalStruct` |
Add a `LaxMonoidalStruct` with only the unit morphism `ε` and the tensorator `μ`. This is used in #6307 to provide two different constructors for `LaxMonoidal` that have common `ε` and `μ` but use the tensor of morphisms or the whiskerings.
---
[](https://gitpod.io/from-referrer/)
|
t-category-theory
merge-conflict
WIP
|
21/8 |
Mathlib/Algebra/Category/ModuleCat/Adjunctions.lean,Mathlib/CategoryTheory/Monoidal/Functorial.lean,Mathlib/CategoryTheory/Monoidal/Limits.lean |
3 |
0 |
[] |
nobody |
409-8939 1 year ago |
597-12788 1 year ago |
0-0 0 seconds |
7835 |
shuxuezhuyi author:shuxuezhuyi |
feat(LinearAlgebra/Matrix): `lift` for projective special linear group |
We provide converters to help with the use of "quotient.liftOn" on projective special linear groups.
---
- [x] depends on: #7826
- [x] depends on: #7791
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
awaiting-author
label:t-algebra$ |
52/0 |
Mathlib/LinearAlgebra/Matrix/ProjectiveSpecialLinearGroup.lean |
1 |
3 |
['jcommelin', 'leanprover-community-mathlib4-bot', 'shuxuezhuyi'] |
jcommelin assignee:jcommelin |
409-8938 1 year ago |
429-48797 1 year ago |
1-85757 1 day |
7351 |
shuxuezhuyi author:shuxuezhuyi |
feat(Topology/Algebra/Order): extend function on `Ioo` to `Icc` |
Extend a strictly monotone function defined on an open interval.
---
[](https://gitpod.io/from-referrer/)
|
t-order
merge-conflict
awaiting-author
|
59/0 |
Mathlib.lean,Mathlib/Data/Set/Function.lean,Mathlib/Topology/Algebra/Order/IccExtendFromIoo.lean |
3 |
7 |
['j-loreaux', 'shuxuezhuyi'] |
nobody |
409-8938 1 year ago |
538-58604 1 year ago |
30-30522 30 days |
7227 |
kmill author:kmill |
feat: flexible binders and integration into notation3 |
Introduces `flexibleBinders`, which is an extensible system for binder notations that allow destructuring, bounded domains, and other niceties. Integrates this into `notation3`, and makes `Finset.sum`/`Finset.prod` use it.
---
- [ ] depends on: #6833
[](https://gitpod.io/from-referrer/)
|
t-meta
merge-conflict
WIP
|
1215/131 |
Mathlib.lean,Mathlib/Algebra/BigOperators/Basic.lean,Mathlib/Algebra/BigOperators/Intervals.lean,Mathlib/Algebra/BigOperators/NatAntidiagonal.lean,Mathlib/Mathport/Notation.lean,Mathlib/Util/FlexibleBinders.lean,Mathlib/Util/FlexibleBindersFinset.lean,Mathlib/Util/SyntaxFun.lean,test/FlexibleBinders.lean,test/notation3.lean |
10 |
3 |
['eric-wieser', 'kmill', 'leanprover-community-mathlib4-bot'] |
nobody |
409-8938 1 year ago |
611-76774 1 year ago |
0-0 0 seconds |
7467 |
ADedecker author:ADedecker |
feat: spectrum of X →ᵇ ℂ is StoneCech X |
---
[](https://gitpod.io/from-referrer/)
|
t-analysis
merge-conflict
WIP
|
121/23 |
Mathlib/Analysis/NormedSpace/Star/BoundedContinuousFunction.lean,Mathlib/Analysis/NormedSpace/Star/GelfandDuality.lean,Mathlib/Topology/ContinuousFunction/Bounded.lean,Mathlib/Topology/ContinuousFunction/Compact.lean |
4 |
1 |
['github-actions'] |
nobody |
409-8938 1 year ago |
570-44350 1 year ago |
0-0 0 seconds |
7427 |
MohanadAhmed author:MohanadAhmed |
Mohanad ahmed/sort eigenvalues abs |
In the file `Analysis.InnerProductSpace.Spectrum` todo notes were left saying:
> TODO Postcompose with a permutation so that these eigenvectors are listed in increasing order of
eigenvalue.
> TODO Postcompose with a permutation so that these eigenvalues are listed in increasing order. -
This is a start in that direction
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict
WIP
|
162/4 |
Mathlib/Analysis/InnerProductSpace/Spectrum.lean,Mathlib/Analysis/NormedSpace/PiLp.lean,Mathlib/LinearAlgebra/Matrix/Spectrum.lean |
3 |
0 |
[] |
nobody |
409-8938 1 year ago |
586-35635 1 year ago |
0-0 0 seconds |
7225 |
jjaassoonn author:jjaassoonn |
some random stuff |
- Consider two commutative rings `R` and `S` and `X` and `(R, S)`-bimodule.
Consider the tensor functor `(X ⊗[R] .)` from the category of `R`-modules to the category of `S`-modules and the hom functor `X →ₗ[S] .` from the category of `S`-modules to the category of `R`-modules, they form an adjunction.
- direct limits of modules commute with tensor product
- A proof of 
Three definitions for flatness:
1. in terms of injectiveness
```lean
def Flat.injective : Prop :=
∀ ⦃N N' : ModuleCat.{u} R⦄ (L : N ⟶ N'),
Function.Injective L → Function.Injective ((tensorRight (ModuleCat.of R M)).map L)
```
2. in terms of ideals
```lean
def Flat.ideal : Prop :=
∀ (I : Ideal R), Function.Injective (TensorProduct.lift ((lsmul R M).comp I.subtype))
```
3. in terms of finitely generated ideal
```lean
def Flat.fg_ideal : Prop :=
∀ ⦃I : Ideal R⦄ (_ : I.FG), Function.Injective (TensorProduct.lift ((lsmul R M).comp I.subtype))
```
and they are all equivalent:
```lean
lemma tfae : List.TFAE
[ Flat.injective R M,
Flat.ideal R M,
Flat.fg_ideal R M ] := by
```
The dependencies between these changed files are:
```
Algebra.Module.LinearMap---------------------------------
| |
| |
v v
Algebra.Category.ModuleCat.TensorProduct -----> Algebra.Character
|
|
|
v
Algebra.DirectLimitAndTensorProduct -------------> RingTheory.Flat
```
to prove equivalence of other definitions, e.g. exact functor, tor, etc should be easier with this because the proof is will be categorical
---
-------------
Some other stuff not about flatness
1. If $S$ is a submonoid and $I$ is maximally disjoint from $S$ then $I$ is prime
2. if $\mathfrak p$ is a minimal prime, then $x \in \mathfrak p$ implies that $x$ is a zero divisor
3. Noetherian rings has only finitely many minimal ideals
4. One version of [the prime avoidance lemma](https://en.wikipedia.org/wiki/Prime_avoidance_lemma): if $E$ is an addsubgroup of a ring and is mutiplicatively closed, and $\mathfrak p_i$ is some prime ideals, then not being any subset of the individual prime ideal implies that not being a subset of their union
----------
[](https://gitpod.io/from-referrer/)
|
merge-conflict |
1828/16 |
Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/TensorProduct.lean,Mathlib/Algebra/Character.lean,Mathlib/Algebra/DirectLimitAndTensorProduct.lean,Mathlib/Algebra/Module/LinearMap.lean,Mathlib/AlgebraicGeometry/PrimeSpectrum/Basic.lean,Mathlib/AlgebraicGeometry/PrimeSpectrum/Noetherian.lean,Mathlib/CategoryTheory/Functor/Fin.lean,Mathlib/CategoryTheory/ShortExactSequence.lean,Mathlib/RingTheory/Flat.lean,Mathlib/RingTheory/Ideal/Basic.lean,Mathlib/RingTheory/Ideal/MinimalPrime.lean,Mathlib/RingTheory/Ideal/PrimeAvoidance.lean |
13 |
6 |
['eric-wieser', 'jjaassoonn'] |
nobody |
409-8938 1 year ago |
602-74243 1 year ago |
0-0 0 seconds |
7932 |
eric-wieser author:eric-wieser |
refactor(Algebra/TrivSqZeroExt): replace with a structure |
This is dogfooding my claim that "one-field structures are the lesser evil in Lean 4".
This runs into the `simp [(stupid_parens)]` bug; or rather, a particular nasty instance of it where the offending simp call is inside `@[simps]`.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
awaiting-CI
merge-conflict
label:t-algebra$ |
155/73 |
Mathlib/Algebra/DualNumber.lean,Mathlib/Algebra/TrivSqZeroExt.lean,Mathlib/Logic/Equiv/TransferInstance.lean,Mathlib/Topology/Instances/TrivSqZeroExt.lean |
4 |
1 |
['github-actions'] |
nobody |
409-8938 1 year ago |
430-76042 1 year ago |
0-0 0 seconds |
7909 |
mcdoll author:mcdoll |
fix(Tactic/Continuity): remove npowRec and add new tag for Continuous.pow |
---
[](https://gitpod.io/from-referrer/)
|
t-topology
t-meta
merge-conflict
WIP
|
14/9 |
Mathlib/Tactic/Continuity.lean,Mathlib/Topology/Category/TopCat/Limits/Basic.lean,test/Continuity.lean |
3 |
2 |
['eric-wieser'] |
nobody |
409-8938 1 year ago |
684-35379 1 year ago |
0-72515 20 hours |
7962 |
eric-wieser author:eric-wieser |
feat: `DualNumber (Quaternion R)` as a `CliffordAlgebra` |
This provides a clifford algebra isomorphic to the dual quaternions
---
- [x] depends on: #7934
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
WIP
label:t-algebra$ |
307/7 |
Mathlib/Algebra/DualNumber.lean,Mathlib/Algebra/QuaternionBasis.lean,Mathlib/LinearAlgebra/CliffordAlgebra/Equivs.lean |
3 |
16 |
['github-actions', 'leanprover-community-mathlib4-bot'] |
nobody |
409-8938 1 year ago |
420-73927 1 year ago |
0-0 0 seconds |
6580 |
adomani author:adomani |
chore: `move_add`-driven replacements |
This PR accompanies #6576 and uses `move_add/mul` to simplify/streamline a selection of proofs.
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict
awaiting-author
|
12/13 |
Counterexamples/Monic_nonRegular.lean,Mathlib/Algebra/Associated.lean,Mathlib/Data/Polynomial/RingDivision.lean,Mathlib/LinearAlgebra/QuadraticForm/Basic.lean |
4 |
0 |
[] |
nobody |
409-8938 1 year ago |
525-83770 1 year ago |
0-0 0 seconds |
6630 |
MohanadAhmed author:MohanadAhmed |
feat: Reduced Spectral Theorem |
For A hermitian matrix $A : n \times n$ with rank $A.rank \leq n$, we can eliminate the zero eigenvalues and their corresponding eigenvectors from the (alternate) spectral theorem. As such the matrix $A$ can be written as: $$A = V₁ D V₁ᴴ$$ where
- $V₁$ : $n \times r$ is the matrix of eigenvector with non-zero associated eigenvalues.
- $D$ is $r \times r$ is the diagonal matrix containing only non-zero eigenvalues on its main diagonal.
with $r = A.rank$ being the rank of the matrix
Towards that goal we make several equivalence definitions:
- `{i // hA.eigenvalues i ≠ 0} ≃ Fin (A.rank)` the set of non-zero eigenvalues can be indexed by the numbers from 0 to (r - 1).
- `{i // ¬ hA.eigenvalues i ≠ 0} ≃ Fin (n - A.rank)` the set of non-zero eigenvalues can be indexed by the numbers from 0 to (n - r - 1).
- `{i // hA.eigenvalues i ≠ 0} ⊕ {i // ¬hA.eigenvalues i ≠ 0} ≃ n`: the index set of the matrix (together with the associated eigenvector matrix and eigenvalues matrix ) can be partitioned into two complement groups the ones corresponding to non-zero eigenvalues and the ones corresponding to zero eigenvalues.
- We can then put the previous definitions together to obtain a: `Fin (A.rank) ⊕ Fin (Fintype.card n - A.rank) ≃ n`
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
WIP
label:t-algebra$ |
31/0 |
Mathlib/LinearAlgebra/Matrix/Spectrum.lean |
1 |
0 |
[] |
nobody |
409-8938 1 year ago |
420-74055 1 year ago |
0-0 0 seconds |
6930 |
kmill author:kmill |
feat: `resynth_instances` tactic for resynthesizing instances in the goal or local context |
This tactic can be useful for debugging non-canonical instances or for fixing up goals and hypotheses after using the `classical` tactic.
---
[](https://gitpod.io/from-referrer/)
|
t-meta
merge-conflict
WIP
|
327/0 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/ResynthInstances.lean,test/ResynthInstances.lean |
4 |
0 |
[] |
nobody |
409-8938 1 year ago |
739-69361 2 years ago |
0-0 0 seconds |
7713 |
RemyDegenne author:RemyDegenne |
feat: add_left/right_inj for measures |
`μ + ν₁ = μ + ν₂ ↔ ν₁ = ν₂`, and similarly on the right. This is not true in general for measures, but is true when `μ` is mutually singular with the two other measures or when `μ` is finite.
---
[](https://gitpod.io/from-referrer/)
|
t-measure-probability
merge-conflict
awaiting-author
|
53/1 |
Mathlib/MeasureTheory/Measure/MutuallySingular.lean,lean-toolchain |
2 |
6 |
['RemyDegenne', 'digama0', 'eric-wieser', 'fpvandoorn'] |
nobody |
409-8938 1 year ago |
683-14778 1 year ago |
0-62955 17 hours |
7601 |
digama0 author:digama0 |
feat: ring hom support in `ring` |
As [requested on Zulip](https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/aroots/near/395750055). Adds support for distributing ring morphisms in `ring`:
```lean
example (p : ℤ[X]) (r : ℤ) : C (2 * r) * p = C r * p + C r * p := by ring
```
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-meta
merge-conflict
awaiting-author
label:t-algebra$ |
257/48 |
Mathlib/Tactic/Ring/Basic.lean,test/linear_combination.lean,test/ring.lean |
3 |
1 |
['eric-wieser'] |
nobody |
409-8938 1 year ago |
466-19930 1 year ago |
0-0 0 seconds |
6931 |
urkud author:urkud |
refactor(Analysis/Normed*): use `RingHomIsometric` for `*.norm_cast` |
---
I don't understand why linter fails.
[](https://gitpod.io/from-referrer/)
|
t-analysis
merge-conflict
help-wanted
|
78/68 |
Mathlib/Analysis/LocallyConvex/ContinuousOfBounded.lean,Mathlib/Analysis/Normed/Field/Basic.lean,Mathlib/Analysis/Normed/Group/Basic.lean,Mathlib/Analysis/NormedSpace/Basic.lean,Mathlib/Analysis/NormedSpace/Exponential.lean,Mathlib/Analysis/NormedSpace/Spectrum.lean,Mathlib/Analysis/RCLike/Basic.lean,Mathlib/NumberTheory/NumberField/Embeddings.lean |
8 |
0 |
[] |
nobody |
409-8938 1 year ago |
430-76042 1 year ago |
0-0 0 seconds |
7615 |
eric-wieser author:eric-wieser |
chore(LinearAlgebra/Basic): generalize compatibleMaps to semilinear maps |
Spotted while reviewing #7611
---
- [x] depends on: #7611
[](https://gitpod.io/from-referrer/)
|
t-algebra
awaiting-CI
easy
merge-conflict
label:t-algebra$ |
9/33 |
Mathlib/LinearAlgebra/Basic.lean |
1 |
1 |
['leanprover-community-mathlib4-bot'] |
nobody |
409-8938 1 year ago |
430-76042 1 year ago |
0-0 0 seconds |
6777 |
adomani author:adomani |
chore(Co*variantClass): replace eta-expanded (· * ·), (· + ·), (· ≤ ·), (· < ·) |
Replace `CovariantClass X X (· * ·) (· ≤ ·)` with -> `CovariantClass X X HMul.hMul LE.le` and similarly for `HAdd`, `LT`, `Contravariant`.
This PR is inspired by [Issue #6646](https://github.com/leanprover-community/mathlib4/issues/6646) and, more specifically, [this comment](https://github.com/leanprover-community/mathlib4/issues/6646#issuecomment-1692792066).
Note that https://github.com/leanprover/lean4/pull/2267 would make this unnecessary
---
```bash
# First sed command:
# the first captured pattern is `Co*variantClass `
# the second captured pattern is ``
# the third captured pattern is `+` or `*`
# the fourth captured pattern is `<` or `≤`
# a match for `Co*variantClass (· ·) (· ·)` becomes
# `Co*variantClass replaceop replaceop`
# Second sed command: similar to the first, but looks for `(Function.swap (· ·))`
sed -i '
s=\(Co[ntra]*variantClass \(..*\) \2 \)(· *\([+*]\) *·) (· *\([<≤]\) *·)=\1replaceop\3 replaceop\4=g
s=\(Co[ntra]*variantClass \(..*\) \2 \)(\([Functio\.swap ]*\)(· *\([+*]\) *·)) (· *\([<≤]\) *·)=\1(\3replaceop\4) replaceop\5=g
s=replaceop+=HAdd.hAdd=g
s=replaceop\*=HMul.hMul=g
s=replaceop<=LT.lt=g
s=replaceop≤=LE.le=g
s=\(Co[ntra]*variantClass N N\) (· \* ·) r=\1 HMul.hMul r=g
s=\(Co[ntra]*variantClass N N (swap μ)\) (· ≤ ·)=\1 LE.le=g
s=\(Co[ntra]*variantClass N N\) (swap (· \* ·)) r=\1 (swap HMul.hMul) r=g
s=\(CovariantClass (Filter α) (Filter α)\) (· / ·) (· ≤ ·)=\1 HDiv.hDiv LE.le=g
s=\(CovariantClass (Filter α) (Filter α)\) (swap (· / ·)) (· ≤ ·)=\1 (swap HDiv.hDiv) LE.le=g
s=\(Co[ntra]*variantClass .* (fun x y .> . \* .)\) (· ≤ ·)=\1 LE.le=g
s=\(Co[ntra]*variantClass .* (fun x y .> . \* .)\) (· < ·)=\1 LT.lt=g
s=\(Co[ntra]*variantClass [^}]*\) (· ≤ ·)=\1 LE.le=g
s=\(CovariantClass .* (Filter β)\) (· • ·) LE.le=\1 HSMul.hSMul LE.le=g
' $(git ls-files '*.lean')
```
[](https://gitpod.io/from-referrer/)
|
merge-conflict |
703/678 |
Counterexamples/ZeroDivisorsInAddMonoidAlgebras.lean,Mathlib/Algebra/BigOperators/Basic.lean,Mathlib/Algebra/Bounds.lean,Mathlib/Algebra/CovariantAndContravariant.lean,Mathlib/Algebra/DirectSum/Internal.lean,Mathlib/Algebra/Group/UniqueProds.lean,Mathlib/Algebra/GroupPower/Order.lean,Mathlib/Algebra/MonoidAlgebra/Degree.lean,Mathlib/Algebra/Order/Archimedean.lean,Mathlib/Algebra/Order/Group/Abs.lean,Mathlib/Algebra/Order/Group/Defs.lean,Mathlib/Algebra/Order/Group/DenselyOrdered.lean,Mathlib/Algebra/Order/Group/MinMax.lean,Mathlib/Algebra/Order/Group/OrderIso.lean,Mathlib/Algebra/Order/Hom/Monoid.lean,Mathlib/Algebra/Order/Interval.lean,Mathlib/Algebra/Order/Kleene.lean,Mathlib/Algebra/Order/LatticeGroup.lean,Mathlib/Algebra/Order/Module.lean,Mathlib/Algebra/Order/Monoid/Basic.lean,Mathlib/Algebra/Order/Monoid/Cancel/Defs.lean,Mathlib/Algebra/Order/Monoid/Canonical/Defs.lean,Mathlib/Algebra/Order/Monoid/Defs.lean,Mathlib/Algebra/Order/Monoid/Lemmas.lean,Mathlib/Algebra/Order/Monoid/MinMax.lean,Mathlib/Algebra/Order/Monoid/NatCast.lean,Mathlib/Algebra/Order/Monoid/OrderDual.lean,Mathlib/Algebra/Order/Monoid/Prod.lean,Mathlib/Algebra/Order/Monoid/WithTop.lean,Mathlib/Algebra/Order/Monoid/WithZero/Basic.lean,Mathlib/Algebra/Order/Monoid/WithZero/Defs.lean,Mathlib/Algebra/Order/Nonneg/Ring.lean,Mathlib/Algebra/Order/Pointwise.lean,Mathlib/Algebra/Order/Positive/Ring.lean,Mathlib/Algebra/Order/Ring/Canonical.lean,Mathlib/Algebra/Order/Ring/Defs.lean,Mathlib/Algebra/Order/Ring/Lemmas.lean,Mathlib/Algebra/Order/Sub/Basic.lean,Mathlib/Algebra/Order/Sub/Canonical.lean,Mathlib/Algebra/Order/Sub/Defs.lean,Mathlib/Algebra/Order/WithZero.lean,Mathlib/Algebra/Parity.lean,Mathlib/Algebra/Star/Order.lean,Mathlib/Algebra/Tropical/Basic.lean,Mathlib/Analysis/Normed/Order/Lattice.lean,Mathlib/Data/DFinsupp/Lex.lean,Mathlib/Data/DFinsupp/Order.lean,Mathlib/Data/Finset/Fold.lean,Mathlib/Data/Finsupp/Lex.lean,Mathlib/Data/Finsupp/Order.lean,Mathlib/Data/List/BigOperators/Basic.lean,Mathlib/Data/List/BigOperators/Lemmas.lean,Mathlib/Data/Multiset/Basic.lean,Mathlib/Data/Nat/Cast/Order.lean,Mathlib/Data/PNat/Basic.lean,Mathlib/Data/Real/ENNReal.lean,Mathlib/Data/Real/NNReal.lean,Mathlib/Data/Set/Semiring.lean,Mathlib/Data/Sign.lean,Mathlib/MeasureTheory/Function/LpOrder.lean,Mathlib/MeasureTheory/Function/SimpleFuncDenseLp.lean,Mathlib/MeasureTheory/Measure/MeasureSpace.lean,Mathlib/MeasureTheory/Measure/VectorMeasure.lean,Mathlib/Order/ConditionallyCompleteLattice/Group.lean,Mathlib/Order/Filter/Basic.lean,Mathlib/Order/Filter/Pointwise.lean,Mathlib/Probability/Martingale/Basic.lean,Mathlib/Probability/Process/Stopping.lean,Mathlib/RingTheory/GradedAlgebra/Basic.lean,Mathlib/SetTheory/Cardinal/Basic.lean,Mathlib/SetTheory/Game/Basic.lean,Mathlib/SetTheory/Game/PGame.lean,Mathlib/SetTheory/Ordinal/Arithmetic.lean,Mathlib/SetTheory/Ordinal/Basic.lean,Mathlib/SetTheory/Ordinal/NaturalOps.lean,Mathlib/Tactic/GCongr/Core.lean,Mathlib/Tactic/Positivity/Basic.lean,Mathlib/Topology/ContinuousFunction/Algebra.lean,lean-toolchain,test/Recall.lean,test/propose.lean |
81 |
36 |
['adomani', 'alreadydone', 'digama0', 'eric-wieser', 'ericrbg', 'jcommelin', 'leanprover-bot', 'sgouezel'] |
nobody |
409-8938 1 year ago |
430-76042 1 year ago |
35-56459 35 days |
7875 |
astrainfinita author:astrainfinita |
chore: make `SMulCommClass A A B` and `SMulCommClass A B B` higher priority |
---
[](https://gitpod.io/from-referrer/)
|
slow-typeclass-synthesis
t-algebra
merge-conflict
label:t-algebra$ |
54/48 |
Mathlib/Algebra/Algebra/Basic.lean,Mathlib/Algebra/Algebra/NonUnitalSubalgebra.lean,Mathlib/Algebra/DirectSum/Algebra.lean,Mathlib/Algebra/Group/Action/Defs.lean,Mathlib/Algebra/Group/Subgroup/Actions.lean,Mathlib/Algebra/Lie/NonUnitalNonAssocAlgebra.lean,Mathlib/Algebra/Module/LinearMap/End.lean,Mathlib/Algebra/MonoidAlgebra/Basic.lean,Mathlib/Algebra/MvPolynomial/Basic.lean,Mathlib/Algebra/Ring/CentroidHom.lean,Mathlib/Algebra/Ring/Subring/Basic.lean,Mathlib/Algebra/Ring/Subsemiring/Basic.lean,Mathlib/Algebra/Star/NonUnitalSubalgebra.lean,Mathlib/Analysis/Complex/UnitDisc/Basic.lean,Mathlib/Analysis/NormedSpace/lpSpace.lean,Mathlib/Data/Matrix/Basic.lean,Mathlib/GroupTheory/GroupAction/Prod.lean,Mathlib/GroupTheory/GroupAction/Ring.lean,Mathlib/GroupTheory/GroupAction/SubMulAction.lean,Mathlib/GroupTheory/MonoidLocalization.lean,Mathlib/GroupTheory/Submonoid/Center.lean,Mathlib/LinearAlgebra/PiTensorProduct.lean,Mathlib/RingTheory/Ideal/Quotient.lean,Mathlib/RingTheory/TensorProduct/Basic.lean,Mathlib/Topology/ContinuousFunction/ContinuousMapZero.lean,Mathlib/Topology/ContinuousFunction/StoneWeierstrass.lean,Mathlib/Topology/ContinuousFunction/ZeroAtInfty.lean |
27 |
15 |
['Parcly-Taxel', 'astrainfinita', 'jcommelin', 'leanprover-bot'] |
nobody |
409-8938 1 year ago |
430-76042 1 year ago |
1-47913 1 day |
6791 |
eric-wieser author:eric-wieser |
refactor: Use flat structures for morphisms |
This restores the symmetry we had in Lean3, where we had `MonoidHom.mk f one mul` not `MonoidHom.mk (OneHom.mk f one) mul`, and `f.toFun` wasn't notation for `f.toMulHom.toFun`.
The nesting provided by the previous inheritance is useless to us in the face of `MonoidHomClass.toMonoidHom`, which completely eta-expands the structure anyway.
We call the class `FunLikeFlatHack._` because this means the field is called `to_` which uses up less space in the goal view than any alternative.
---
[](https://gitpod.io/from-referrer/)
|
awaiting-CI
merge-conflict
awaiting-author
help-wanted
|
174/201 |
Mathlib/Algebra/Algebra/Equiv.lean,Mathlib/Algebra/Algebra/Hom.lean,Mathlib/Algebra/Category/GroupCat/ZModuleEquivalence.lean,Mathlib/Algebra/Category/GroupWithZeroCat.lean,Mathlib/Algebra/Category/ModuleCat/Presheaf.lean,Mathlib/Algebra/Category/MonCat/Basic.lean,Mathlib/Algebra/Group/Ext.lean,Mathlib/Algebra/Group/Prod.lean,Mathlib/Algebra/Group/UniqueProds.lean,Mathlib/Algebra/Hom/Equiv/Basic.lean,Mathlib/Algebra/Hom/Group/Defs.lean,Mathlib/Algebra/Hom/GroupAction.lean,Mathlib/Algebra/Hom/NonUnitalAlg.lean,Mathlib/Algebra/Hom/Ring/Defs.lean,Mathlib/Algebra/Lie/Basic.lean,Mathlib/Algebra/Module/Equiv.lean,Mathlib/Algebra/Module/LinearMap.lean,Mathlib/Algebra/Order/Hom/Ring.lean,Mathlib/Algebra/Order/Interval.lean,Mathlib/Algebra/Ring/Equiv.lean,Mathlib/Analysis/Normed/Group/SemiNormedGroupCat.lean,Mathlib/Data/FunLike/Basic.lean,Mathlib/Data/Rat/Cast/CharZero.lean,Mathlib/Data/Real/EReal.lean,Mathlib/Data/Real/Sqrt.lean,Mathlib/GroupTheory/FreeAbelianGroup.lean,Mathlib/GroupTheory/MonoidLocalization.lean,Mathlib/LinearAlgebra/Quotient.lean,Mathlib/LinearAlgebra/TensorProduct.lean,Mathlib/RingTheory/RingInvo.lean,Mathlib/Topology/Algebra/Module/Basic.lean,Mathlib/Topology/MetricSpace/Dilation.lean |
32 |
0 |
[] |
nobody |
409-8938 1 year ago |
725-63198 1 year ago |
0-0 0 seconds |
6307 |
yuma-mizuno author:yuma-mizuno |
refactor(CategoryTheory/Monoidal): add whiskering operators |
We introduce whiskering operators. This allows us to introduce a simp-normal form for morphisms in monoidal categories. Rewriting into simp-normal forms is especially useful when combined with the coherence tactic.
---
- [x] depends on: #6420
- [x] depends on: #8191
- [x] depends on: #9988
- [x] depends on: #9991
- [x] depends on: #9995
- [x] depends on: #10061
- [x] depends on: #10078
- [x] depends on: #10898
- [x] depends on: #10912
- [x] depends on: #11223
[](https://gitpod.io/from-referrer/)
|
t-category-theory
merge-conflict
awaiting-author
|
325/280 |
Mathlib/Algebra/Category/ModuleCat/Adjunctions.lean,Mathlib/CategoryTheory/Bicategory/End.lean,Mathlib/CategoryTheory/Closed/Ideal.lean,Mathlib/CategoryTheory/Monoidal/Category.lean,Mathlib/CategoryTheory/Monoidal/Center.lean,Mathlib/CategoryTheory/Monoidal/Free/Basic.lean,Mathlib/CategoryTheory/Monoidal/Free/Coherence.lean,Mathlib/CategoryTheory/Monoidal/Functor.lean,Mathlib/CategoryTheory/Monoidal/FunctorCategory.lean,Mathlib/CategoryTheory/Monoidal/Limits.lean,Mathlib/CategoryTheory/Monoidal/Mon_.lean,Mathlib/CategoryTheory/Monoidal/NaturalTransformation.lean,Mathlib/CategoryTheory/Monoidal/Opposite.lean,Mathlib/CategoryTheory/Monoidal/Transport.lean,test/CategoryTheory/Coherence.lean |
15 |
38 |
['eric-wieser', 'github-actions', 'grunweg', 'jcommelin', 'kim-em', 'leanprover-community-mathlib4-bot', 'yuma-mizuno'] |
nobody |
409-8937 1 year ago |
424-21766 1 year ago |
0-0 0 seconds |
6079 |
eric-wieser author:eric-wieser |
fix: deduplicate variables |
`variables {A} [Ring A]` meant "update the binder of `A`" in Lean 3, but now means "create a duplicate variable called `A`" (or at least, does so when inspecting the state within the variables line).
This removes a number of porting notes that were stumbling over this behavior.
[Related Zulip thread](https://leanprover.zulipchat.com/#narrow/stream/270676-lean4/topic/unexpected.20.60variable.60.20behaviour.3F/near/360154080)
---
[](https://gitpod.io/from-referrer/)
|
awaiting-CI
merge-conflict
|
1012/443 |
Archive/Wiedijk100Theorems/CubingACube.lean,Mathlib/Algebra/Category/ModuleCat/Adjunctions.lean,Mathlib/Algebra/CharP/Basic.lean,Mathlib/Algebra/CovariantAndContravariant.lean,Mathlib/Algebra/DirectLimit.lean,Mathlib/Algebra/DirectSum/Finsupp.lean,Mathlib/Algebra/DirectSum/Module.lean,Mathlib/Algebra/GradedMonoid.lean,Mathlib/Algebra/Group/Pi.lean,Mathlib/Algebra/GroupPower/Basic.lean,Mathlib/Algebra/GroupPower/Lemmas.lean,Mathlib/Algebra/Hom/Aut.lean,Mathlib/Algebra/Hom/Equiv/Basic.lean,Mathlib/Algebra/Hom/Group.lean,Mathlib/Algebra/Homology/HomologicalComplex.lean,Mathlib/Algebra/Homology/HomotopyCategory.lean,Mathlib/Algebra/Homology/ImageToKernel.lean,Mathlib/Algebra/Homology/ShortComplex/LeftHomology.lean,Mathlib/Algebra/IndicatorFunction.lean,Mathlib/Algebra/Jordan/Basic.lean,Mathlib/Algebra/Lie/Classical.lean,Mathlib/Algebra/Lie/Subalgebra.lean,Mathlib/Algebra/Lie/Submodule.lean,Mathlib/Algebra/Lie/TensorProduct.lean,Mathlib/Algebra/Module/Injective.lean,Mathlib/Algebra/Module/LinearMap.lean,Mathlib/Algebra/Module/Submodule/Basic.lean,Mathlib/Algebra/MonoidAlgebra/Basic.lean,Mathlib/Algebra/MonoidAlgebra/Grading.lean,Mathlib/Algebra/Order/CompleteField.lean,Mathlib/Algebra/Order/Pi.lean,Mathlib/Algebra/Order/Ring/Lemmas.lean,Mathlib/Algebra/Ring/Equiv.lean,Mathlib/Algebra/SMulWithZero.lean,Mathlib/Algebra/Star/Module.lean,Mathlib/Algebra/Support.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Point.lean,Mathlib/AlgebraicGeometry/Morphisms/RingHomProperties.lean,Mathlib/AlgebraicGeometry/ProjectiveSpectrum/Scheme.lean,Mathlib/AlgebraicGeometry/StructureSheaf.lean,Mathlib/AlgebraicTopology/DoldKan/Decomposition.lean,Mathlib/AlgebraicTopology/MooreComplex.lean,Mathlib/Analysis/Calculus/ContDiff.lean,Mathlib/Analysis/Calculus/FormalMultilinearSeries.lean,Mathlib/Analysis/Calculus/LocalExtr.lean,Mathlib/Analysis/Calculus/TangentCone.lean,Mathlib/Analysis/Convex/Basic.lean,Mathlib/Analysis/Convex/Combination.lean,Mathlib/Analysis/Convex/Extreme.lean,Mathlib/Analysis/Convex/Function.lean,Mathlib/Analysis/Convex/Hull.lean,Mathlib/Analysis/Convex/Independent.lean,Mathlib/Analysis/Convex/Intrinsic.lean,Mathlib/Analysis/Convex/Join.lean,Mathlib/Analysis/Convex/Quasiconvex.lean,Mathlib/Analysis/Convex/Segment.lean,Mathlib/Analysis/Convex/Star.lean,Mathlib/Analysis/Convex/Uniform.lean,Mathlib/Analysis/Convolution.lean,Mathlib/Analysis/Fourier/RiemannLebesgueLemma.lean,Mathlib/Analysis/InnerProductSpace/Calculus.lean,Mathlib/Analysis/LocallyConvex/AbsConvex.lean,Mathlib/Analysis/LocallyConvex/BalancedCoreHull.lean,Mathlib/Analysis/LocallyConvex/Basic.lean,Mathlib/Analysis/LocallyConvex/Bounded.lean,Mathlib/Analysis/LocallyConvex/WithSeminorms.lean,Mathlib/Analysis/Normed/Field/Basic.lean,Mathlib/Analysis/Normed/Group/AddCircle.lean,Mathlib/Analysis/Normed/Group/Hom.lean,Mathlib/Analysis/Normed/Group/Seminorm.lean,Mathlib/Analysis/NormedSpace/Completion.lean,Mathlib/Analysis/NormedSpace/LinearIsometry.lean,Mathlib/Analysis/NormedSpace/Multilinear.lean,Mathlib/Analysis/NormedSpace/OperatorNorm.lean,Mathlib/Analysis/ODE/PicardLindelof.lean,Mathlib/Analysis/Seminorm.lean,Mathlib/CategoryTheory/Action.lean,Mathlib/CategoryTheory/Bicategory/LocallyDiscrete.lean,Mathlib/CategoryTheory/Bicategory/NaturalTransformation.lean,Mathlib/CategoryTheory/Closed/Ideal.lean,Mathlib/CategoryTheory/ConcreteCategory/UnbundledHom.lean,Mathlib/CategoryTheory/Core.lean,Mathlib/CategoryTheory/Endofunctor/Algebra.lean,Mathlib/CategoryTheory/Enriched/Basic.lean,Mathlib/CategoryTheory/EssentialImage.lean,Mathlib/CategoryTheory/FullSubcategory.lean,Mathlib/CategoryTheory/Functor/Category.lean,Mathlib/CategoryTheory/Limits/Fubini.lean,Mathlib/CategoryTheory/Limits/HasLimits.lean,Mathlib/CategoryTheory/Limits/Preserves/Shapes/Kernels.lean,Mathlib/CategoryTheory/Limits/Shapes/BinaryProducts.lean,Mathlib/CategoryTheory/Limits/Shapes/Biproducts.lean,Mathlib/CategoryTheory/Limits/Shapes/Equalizers.lean,Mathlib/CategoryTheory/Limits/Shapes/Images.lean,Mathlib/CategoryTheory/Limits/Shapes/WidePullbacks.lean,Mathlib/CategoryTheory/Linear/LinearFunctor.lean,Mathlib/CategoryTheory/Localization/Construction.lean,Mathlib/CategoryTheory/Monoidal/Braided.lean,Mathlib/CategoryTheory/Monoidal/CommMon_.lean,Mathlib/CategoryTheory/Monoidal/Discrete.lean |
302 |
1 |
['timotree3'] |
nobody |
409-8937 1 year ago |
430-76042 1 year ago |
0-0 0 seconds |
6002 |
slerpyyy author:slerpyyy |
feat(Analysis.SpecialFunctions.Gaussian): add `integrable_fun_mul_exp_neg_mul_sq` |
If `f : ℝ → ℝ` is bounded by a polynomial, `fun x : ℝ => f x * exp (-b * x ^ 2)` is integrable.
---
[](https://gitpod.io/from-referrer/)
|
t-analysis
merge-conflict
awaiting-author
|
26/0 |
Mathlib/Analysis/SpecialFunctions/Gaussian.lean |
1 |
3 |
['ocfnash', 'slerpyyy', 'urkud'] |
nobody |
409-8937 1 year ago |
673-84934 1 year ago |
9-67365 9 days |
4871 |
j-loreaux author:j-loreaux |
feat: define the additive submonoid of positive elements in a star ordered ring |
This file defines the `AddSubmonoid` of nonegative elements `StarOrderedRing.positive R` in a star ordered ring `R` with carrier `{ x : R | 0 ≤ x }` (in fact, the definition only requires `OrderedAddCommMonoid R` to allow for other use cases, but it is primarily intended for `StarOrderedRing R`). Equivalently, this is the `AddSubmonoid` generated by the elements of the form `star s * s`. Even though this technically corresponds to the nonnegative elements, the "positive" terminology is standard throughout the literature (at least in C⋆-algebra theory and operator theory), so we choose to prefer that.
The advantage of using this over other definitions of positivity is that it allows us to unify several different concepts under a single umbrella. For example, one might be tempted to consider the collection of bounded linear operators on an Hilbert space and define positivity as `∀ x, 0 ≤ ⟪T x, x⟫`, but this doesn't generalize nicely to C⋆-algebras. Alternatively, one could define positivity as those self-adjoint elements with nonnegative spectrum, but this requires the algebra to be unital. Our definition herein conveniently sidesteps these issues.
---
Note: I declared the `AddMonoidWithOne` and `AddGroupWithOne` instances for `selfAdjoint R` separately because it made the proof of the latter easier.
- [x] depends on: #6229
- [x] depends on: #10209
[](https://gitpod.io/from-referrer/)
|
t-algebra
awaiting-CI
merge-conflict
label:t-algebra$ |
216/12 |
Mathlib.lean,Mathlib/Algebra/Order/Ring/CharZero.lean,Mathlib/Algebra/Star/Order.lean,Mathlib/Algebra/Star/Positive.lean,Mathlib/Algebra/Star/SelfAdjoint.lean,Mathlib/GroupTheory/Submonoid/Operations.lean |
6 |
28 |
['eric-wieser', 'j-loreaux', 'leanprover-community-mathlib4-bot'] |
nobody |
409-8937 1 year ago |
430-76042 1 year ago |
5-55287 5 days |
6491 |
eric-wieser author:eric-wieser |
chore(Mathlib/Algebra/Hom/GroupAction): add `SMulHomClass.comp_smul` |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
label:t-algebra$ |
24/10 |
Mathlib/Algebra/Hom/GroupAction.lean |
1 |
0 |
[] |
nobody |
409-8937 1 year ago |
430-76042 1 year ago |
83-76369 83 days |
6195 |
eric-wieser author:eric-wieser |
chore(RingTheory/TensorProduct): golf the `mul` definition |
---
- [x] depends on: #6211
- [x] depends on: #6187
[](https://gitpod.io/from-referrer/)
Strangely this causes a timeout downstream
|
t-algebra
awaiting-CI
merge-conflict
label:t-algebra$ |
4/29 |
Mathlib/RingTheory/TensorProduct.lean |
1 |
1 |
['leanprover-community-mathlib4-bot'] |
nobody |
409-8937 1 year ago |
430-76042 1 year ago |
0-0 0 seconds |
5912 |
ADedecker author:ADedecker |
feat(Analysis.Distribution.ContDiffMapSupportedIn): space of smooth maps with support in a fixed compact |
---
[](https://gitpod.io/from-referrer/)
|
t-analysis
merge-conflict
WIP
|
513/13 |
Mathlib.lean,Mathlib/Analysis/Distribution/ContDiffMapSupportedIn.lean,Mathlib/Analysis/LocallyConvex/WithSeminorms.lean,Mathlib/Analysis/Seminorm.lean,Mathlib/Data/FunLike/Basic.lean,Mathlib/Data/Set/Function.lean,Mathlib/Topology/Algebra/Module/StrongTopology.lean,Mathlib/Topology/ContinuousFunction/Bounded.lean |
8 |
0 |
[] |
nobody |
409-8937 1 year ago |
759-62978 2 years ago |
0-0 0 seconds |
6268 |
eric-wieser author:eric-wieser |
Fixups to #3838 |
This is an attempt to make #3838 universe polymorphic
---
[](https://gitpod.io/from-referrer/)
* Depends on #6271
* Depends on #8876 |
merge-conflict
WIP
|
186/107 |
Mathlib/Control/Random.lean,Mathlib/Tactic/SlimCheck.lean,Mathlib/Testing/SlimCheck/Functions.lean,Mathlib/Testing/SlimCheck/Gen.lean,Mathlib/Testing/SlimCheck/Sampleable.lean,Mathlib/Testing/SlimCheck/Testable.lean,test/slim_check.lean |
7 |
10 |
['github-actions', 'kim-em'] |
nobody |
409-8937 1 year ago |
635-40804 1 year ago |
0-0 0 seconds |
6590 |
mcdoll author:mcdoll |
feat: composition of LinearPMaps |
This PR changes the definition of the composition to allow composition of arbitrary LinearPMaps by restricting the domains appropriately.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
WIP
label:t-algebra$ |
51/7 |
Mathlib/LinearAlgebra/LinearPMap.lean,lean-toolchain |
2 |
3 |
['ADedecker', 'digama0', 'mcdoll'] |
nobody |
409-8937 1 year ago |
683-15544 1 year ago |
3-26416 3 days |
6328 |
FR-vdash-bot author:FR-vdash-bot |
chore: make some instance about `Sub...Class` lower priority |
Many similar instances have been marked as lower priority. I'd like to see if this would make things faster.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
awaiting-CI
merge-conflict
WIP
label:t-algebra$ |
14/14 |
Mathlib/RingTheory/NonUnitalSubsemiring/Basic.lean,Mathlib/RingTheory/Subsemiring/Basic.lean,lean-toolchain |
3 |
1 |
['digama0'] |
nobody |
409-8937 1 year ago |
683-15545 1 year ago |
0-0 0 seconds |
6210 |
MohanadAhmed author:MohanadAhmed |
feat(Data/IsROrC/Basic): add a `StarOrderedRing` instance |
This PR implements a suggestion by @urkud on [Zulip thread](https://leanprover.zulipchat.com/#narrow/stream/113488-general/topic/PartialOrder.20and.20StarOrderedRing.20on.20IsROrC) on how to get a `StarOrderedRing` on the `IsROrC` class. In that discussion the suggested step were:
1. Add PartialOrder K to the list of extends and add le_iff_re_im : z ≤ w ↔ re z ≤ re w ∧ im z = im w to the list of axioms.
2. Prove StarOrderedRing instance for any IsROrC.
3. Add (almost trivial) le_iff_re_im proofs to IsROrC instances for real and complex numbers.
This PR does exactly these three steps
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-analysis
merge-conflict
WIP
label:t-algebra$ |
25/24 |
Mathlib/Analysis/Complex/Basic.lean,Mathlib/Analysis/SpecialFunctions/Pow/Deriv.lean,Mathlib/Data/Complex/Basic.lean,Mathlib/Data/IsROrC/Basic.lean |
4 |
19 |
['MohanadAhmed', 'eric-wieser', 'j-loreaux'] |
nobody |
409-8937 1 year ago |
760-12074 2 years ago |
0-4269 1 hour |
7076 |
grunweg author:grunweg |
feat: define measure zero subsets of a manifold |
A topological manifold has no canonical measure, but there is a canonical notion of measure zero subsets.
We show that these are closed under subsets and countable unions (hence define a filter, the almost everywhere filter)
and that a closed nowhere dense has empty interior.
This is necessary for stating the general version of Sard's theorem (in finite dimensions), and a first step towards its proof.
This code was written at LftCM 2023. Thanks for @fpvandoorn for mentoring me! :heart:
---
Unresolved questions/looking for feedback
- Is "measure zero" a good name or would "null set" be better? I tend towards the former, but welcome input from a measure theorist (which I'm not).
- What is the correct definition? One could also define "measure zero" using any `IsOpenPosMeasure` on the charted space.
I think all results in this file still hold then, but for applications (e.g., Sard's theorem), this might be too general.
- define custom notation, similar to the a.e. filter on a measure space? (We could include $J$ instead of $\mu$.)
- what's the right syntax for formulas in docstrings --- use LaTeX or backticks? I don't know how to preview the generated docs, the guidelines are a bit ambiguous for me.
|
t-measure-probability
t-differential-geometry
merge-conflict
WIP
|
165/0 |
Mathlib.lean,Mathlib/Geometry/Manifold/MeasureZero.lean,docs/references.bib |
3 |
27 |
['ADedecker', 'github-actions', 'grunweg', 'mo271', 'sgouezel'] |
ADedecker assignee:ADedecker |
409-8937 1 year ago |
448-4748 1 year ago |
43-56043 43 days |
6633 |
adomani author:adomani |
feat(..Polynomial..): `MvPolynomial`s have no zero divisors |
This PR continues #6627, placing the `NoZeroDivisors` instance on `MvPolynomial`s and removing auxiliary intermediate results that are no longer needed.
Affected files:
```
Data/MvPolynomial/Basic.lean
Data/Polynomial/RingDivision.lean
RingTheory/Polynomial/Basic.lean
```
---
- [ ] depends on: #6227 for the `NoZeroDivisors` instance on `AddMonoidAlgebra`s
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
awaiting-author
label:t-algebra$ |
143/57 |
Mathlib/Algebra/MonoidAlgebra/NoZeroDivisors.lean,Mathlib/Data/MvPolynomial/Basic.lean,Mathlib/Data/Polynomial/RingDivision.lean,Mathlib/RingTheory/Polynomial/Basic.lean |
4 |
4 |
['adomani', 'eric-wieser', 'leanprover-community-mathlib4-bot'] |
nobody |
409-8937 1 year ago |
755-56862 2 years ago |
0-19160 5 hours |
6330 |
FR-vdash-bot author:FR-vdash-bot |
chore: make some instance about `Sub...Class` higher priority than `Sub...` |
The opposite direction to #6328.
---
[](https://gitpod.io/from-referrer/)
|
slow-typeclass-synthesis
t-algebra
merge-conflict
WIP
label:t-algebra$ |
123/128 |
Mathlib/Algebra/Algebra/NonUnitalSubalgebra.lean,Mathlib/Algebra/Algebra/Subalgebra/Basic.lean,Mathlib/Algebra/Star/NonUnitalSubalgebra.lean,Mathlib/FieldTheory/IsAlgClosed/Basic.lean,Mathlib/FieldTheory/Subfield.lean,Mathlib/RingTheory/NonUnitalSubring/Basic.lean,Mathlib/RingTheory/NonUnitalSubsemiring/Basic.lean,Mathlib/RingTheory/Polynomial/Quotient.lean,Mathlib/RingTheory/Subring/Basic.lean,Mathlib/RingTheory/Subsemiring/Basic.lean,lean-toolchain |
11 |
13 |
['FR-vdash-bot', 'digama0', 'leanprover-bot'] |
nobody |
409-8937 1 year ago |
467-52427 1 year ago |
0-0 0 seconds |
6993 |
jjaassoonn author:jjaassoonn |
feat : lemmas about `AddMonoidAlgebra.{divOf, modOf}` |
---
- [x] depends on: #7582
- [x] depends on: #8975
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
label:t-algebra$ |
147/3 |
Mathlib/Algebra/MonoidAlgebra/Division.lean,Mathlib/Data/Finsupp/Basic.lean,Mathlib/Data/MvPolynomial/Basic.lean,Mathlib/Data/MvPolynomial/CommRing.lean,Mathlib/Data/MvPolynomial/Division.lean |
5 |
42 |
['YaelDillies', 'alreadydone', 'digama0', 'eric-wieser', 'github-actions', 'jjaassoonn', 'leanprover-community-mathlib4-bot'] |
nobody |
409-8937 1 year ago |
430-76042 1 year ago |
102-21189 102 days |
6403 |
FR-vdash-bot author:FR-vdash-bot |
chore: change instance priorities of `Ordered*` hierarchy |
---
[](https://gitpod.io/from-referrer/)
|
slow-typeclass-synthesis
t-order
t-algebra
merge-conflict
awaiting-author
label:t-algebra$ |
253/79 |
Mathlib/Algebra/Order/CompleteField.lean,Mathlib/Algebra/Order/Field/Canonical/Defs.lean,Mathlib/Algebra/Order/Field/Defs.lean,Mathlib/Algebra/Order/Group/Defs.lean,Mathlib/Algebra/Order/Monoid/Basic.lean,Mathlib/Algebra/Order/Monoid/Canonical/Defs.lean,Mathlib/Algebra/Order/Monoid/Defs.lean,Mathlib/Algebra/Order/Monoid/WithZero/Defs.lean,Mathlib/Algebra/Order/Ring/Canonical.lean,Mathlib/Algebra/Order/Ring/Defs.lean,Mathlib/Algebra/Order/Ring/Star.lean,Mathlib/Algebra/Order/WithZero.lean,Mathlib/Analysis/InnerProductSpace/Orientation.lean,Mathlib/LinearAlgebra/Orientation.lean,Mathlib/RingTheory/HahnSeries.lean,Mathlib/RingTheory/LaurentSeries.lean,Mathlib/Tactic/Positivity/Core.lean,Mathlib/Topology/Algebra/WithZeroTopology.lean |
18 |
39 |
['FR-vdash-bot', 'Vierkantor', 'digama0', 'eric-wieser', 'j-loreaux', 'leanprover-bot'] |
nobody |
409-8937 1 year ago |
467-52407 1 year ago |
13-18399 13 days |
4775 |
thorimur author:thorimur |
feat: `SubExpr` utilities |
This file contains utilities for handling positions in expressions, including folding over subexpressions along with their positions.
---
[](https://gitpod.io/from-referrer/)
|
t-meta
merge-conflict
WIP
|
148/0 |
Mathlib.lean,Mathlib/Lean/SubExpr.lean |
2 |
0 |
[] |
nobody |
409-8937 1 year ago |
829-20253 2 years ago |
0-0 0 seconds |
5133 |
kmill author:kmill |
feat: IntermediateField adjoin syntax for sets of elements |
Adds support for both `F⟮S⟯` and `F⟮α⟯`. The term `x` in `F⟮x⟯` is elaborated, and if it has type `Set _` the first interpretation is used, and otherwise the second is.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
WIP
label:t-algebra$ |
110/55 |
Mathlib/FieldTheory/Adjoin.lean |
1 |
0 |
[] |
nobody |
409-8937 1 year ago |
764-47201 2 years ago |
0-0 0 seconds |
3575 |
Kha author:Kha |
perf: selectively enable precompilation |
---
This is an initial performance test on Linux. TODO:
- [ ] test on macOS and Windows as well
- [ ] adapt caching |
merge-conflict
WIP
|
3/0 |
lakefile.lean |
1 |
21 |
['Kha', 'kim-em', 'leanprover-bot', 'tydeu'] |
nobody |
409-8937 1 year ago |
440-68932 1 year ago |
0-0 0 seconds |
4771 |
thorimur author:thorimur |
feat: Backtrack minimize |
Utilities for backtracking in order to attain a minimum according to some arbitrary notion of size when generating lists of parts and alternatives in alternating fashion. Motivated by minimizing the number of generated subgoals under apply-like actions on the goal.
---
[](https://gitpod.io/from-referrer/)
|
t-meta
merge-conflict
|
482/1 |
Mathlib/Tactic/Backtracking.lean,test/Backtracking.lean |
2 |
0 |
[] |
nobody |
409-8937 1 year ago |
731-28312 2 years ago |
0-0 0 seconds |
4109 |
kim-em author:kim-em |
feat: run library_search when the cursor is at a sorry |
---
[](https://gitpod.io/from-referrer/)
|
t-meta
merge-conflict
|
77/0 |
Mathlib.lean,Mathlib/Data/Nondet/Basic.lean,Mathlib/Tactic/Common.lean,Mathlib/Tactic/LibrarySearch.lean,Mathlib/Util/CodeAction/RunTactic.lean |
5 |
0 |
[] |
nobody |
409-8937 1 year ago |
617-29129 1 year ago |
0-0 0 seconds |
3808 |
kim-em author:kim-em |
feat: #formalize, backed by a choice of LLMs |
This replaces
* https://github.com/leanprover-community/mathlib4/pull/3785, which has essentially been moved to an [independent repository](https://github.com/leanprover-community/llm) and generalised to interface with a choice of OpenAI's GPT, a gpt4all model (running locally via their python binding), or a model compatible with `llama.cpp` (e.g. the 4-bit quantised versions of Meta's LLaMa models).
* https://github.com/leanprover-community/mathlib4/pull/3786, which has been modified slightly but still adds code here in `Mathlib.Tactic.Formalize`.
Typical output:
```
#formalize "There are infinitely many primes numbers ending with a 7."
```
produces:
* GPT4
```
-- /-- There are infinitely many prime numbers ending with a 7. -/
-- theorem infinitely_many_primes_ending_with_7 : ∀ N : Nat, ∃ p, N < p ∧ p.Prime ∧ p % 10 = 7 :=
-- sorry
```
* ggml-gpt4all-j-v1.3-groovy.bin:
```
-- There are infinitely many prime numbers that end with a 7.
```
* 7B/ggml-model-q4_0.bin:
```
-- ∀ p : nat, 7 < 7p + 1 := sorry
-– \end{code}
```
There are other sample outputs in `test/formalize.lean`
If you don't currently have a LLM that the `leanprover-community/llm` project can recognise, when you run `#formalize` you get an error message, which currently reads:
```
Could not find a usable chat bot!
You can try one of the following:
* Obtain an OpenAI API access key at https://platform.openai.com/account/api-keys,
and store it in the environment variable OPENAI_API_KEY.
This will enable you to use ChatGPT.
* Download the GPT4All-J model `https://gpt4all.io/models/ggml-gpt4all-j-v1.3-groovy.bin`,
and put it in either `$HOME/.models/` or `$LLM_MODELS`.
Also install the gpt4all python bindings via `pip3 install pygpt4all`.
* Clone the `llama.cpp` repository from https://github.com/ggerganov/llama.cpp.
Set the environment variable `LLAMA_CPP_HOME` to this repository.
Follow the instructions in the README to produce `7B/ggml-model-q4_0.bin`
starting from the Meta LLaMa weights.
You can store this file at one of
* `$LLAMA_CPP_HOME/models/7B/ggml-model-q4_0.bin`
* `$HOME/.models/7B/ggml-model-q4_0.bin`
* `$LLM_MODELS/7B/ggml-model-q4_0.bin`
```
Currently there are not user-configurable hooks to pick which LLM to use: it checks the conditions described in those bullet points, and takes the first one it finds. (i.e. if you want to use the LLaMa `7B/ggml-model-q4_0.bin`, you have to remove your OpenAI API key!). However a tactic in a downstream project (e.g. mathlib) can specify which interface and model it wants to use, or just call `findChatBot` for the behaviour described in that message.
---
[](https://gitpod.io/from-referrer/)
|
t-meta
merge-conflict
awaiting-author
|
180/0 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Formalize.lean,lake-manifest.json,lakefile.lean,test/formalize.lean |
6 |
2 |
['digama0', 'jcommelin'] |
nobody |
409-8937 1 year ago |
729-12065 1 year ago |
124-45187 124 days |
4127 |
kmill author:kmill |
refactor: create HasAdj class, define Digraph, and generalize some SimpleGraph API |
---
[](https://gitpod.io/from-referrer/)
|
t-combinatorics
merge-conflict
awaiting-author
|
1403/551 |
Mathlib.lean,Mathlib/Combinatorics/Digraph/Basic.lean,Mathlib/Combinatorics/Graph/Classes.lean,Mathlib/Combinatorics/Graph/Dart.lean,Mathlib/Combinatorics/Graph/Hom.lean,Mathlib/Combinatorics/SimpleGraph/AdjMatrix.lean,Mathlib/Combinatorics/SimpleGraph/Basic.lean,Mathlib/Combinatorics/SimpleGraph/Clique.lean,Mathlib/Combinatorics/SimpleGraph/Coloring.lean,Mathlib/Combinatorics/SimpleGraph/Connectivity.lean,Mathlib/Combinatorics/SimpleGraph/DegreeSum.lean,Mathlib/Combinatorics/SimpleGraph/Density.lean,Mathlib/Combinatorics/SimpleGraph/Ends/Defs.lean,Mathlib/Combinatorics/SimpleGraph/Finsubgraph.lean,Mathlib/Combinatorics/SimpleGraph/Hasse.lean,Mathlib/Combinatorics/SimpleGraph/Prod.lean,Mathlib/Combinatorics/SimpleGraph/StronglyRegular.lean,Mathlib/Combinatorics/SimpleGraph/Subgraph.lean |
18 |
0 |
[] |
nobody |
409-8937 1 year ago |
450-6365 1 year ago |
0-0 0 seconds |
5934 |
eric-wieser author:eric-wieser |
feat: port Data.Rat.MetaDefs |
---
[](https://gitpod.io/from-referrer/)
This needs some eyes from people familiar with Qq |
t-meta
merge-conflict
mathlib-port
help-wanted
|
183/0 |
Mathlib.lean,Mathlib/Data/Rat/MetaDefs.lean,test/rat.lean |
3 |
4 |
['eric-wieser', 'gebner'] |
nobody |
409-8937 1 year ago |
578-82326 1 year ago |
0-0 0 seconds |
4960 |
eric-wieser author:eric-wieser |
chore: use `open scoped` |
Earlier versions of mathport did not know about this.
This was done by searching for all `open` commands referencing:
* `Classical`
* `BigOperators`
* `Topology`
* `Pointwise`
---
[](https://gitpod.io/from-referrer/)
|
awaiting-CI
merge-conflict
|
1026/981 |
Mathlib/Algebra/AddTorsor.lean,Mathlib/Algebra/Algebra/Basic.lean,Mathlib/Algebra/Algebra/Equiv.lean,Mathlib/Algebra/Algebra/Hom.lean,Mathlib/Algebra/Algebra/Operations.lean,Mathlib/Algebra/Algebra/Subalgebra/Basic.lean,Mathlib/Algebra/Algebra/Subalgebra/Pointwise.lean,Mathlib/Algebra/Algebra/Subalgebra/Tower.lean,Mathlib/Algebra/Algebra/Tower.lean,Mathlib/Algebra/BigOperators/Associated.lean,Mathlib/Algebra/BigOperators/Basic.lean,Mathlib/Algebra/BigOperators/Fin.lean,Mathlib/Algebra/BigOperators/Finprod.lean,Mathlib/Algebra/BigOperators/Finsupp.lean,Mathlib/Algebra/BigOperators/Intervals.lean,Mathlib/Algebra/BigOperators/NatAntidiagonal.lean,Mathlib/Algebra/BigOperators/Option.lean,Mathlib/Algebra/BigOperators/Order.lean,Mathlib/Algebra/BigOperators/Pi.lean,Mathlib/Algebra/BigOperators/Ring.lean,Mathlib/Algebra/BigOperators/RingEquiv.lean,Mathlib/Algebra/Bounds.lean,Mathlib/Algebra/Category/GroupCat/Biproducts.lean,Mathlib/Algebra/Category/GroupCat/FilteredColimits.lean,Mathlib/Algebra/Category/GroupCat/Injective.lean,Mathlib/Algebra/Category/ModuleCat/Adjunctions.lean,Mathlib/Algebra/Category/ModuleCat/Biproducts.lean,Mathlib/Algebra/Category/Mon/FilteredColimits.lean,Mathlib/Algebra/Category/Ring/Adjunctions.lean,Mathlib/Algebra/Category/Ring/FilteredColimits.lean,Mathlib/Algebra/CharP/Basic.lean,Mathlib/Algebra/CharP/Two.lean,Mathlib/Algebra/DirectLimit.lean,Mathlib/Algebra/DirectSum/Basic.lean,Mathlib/Algebra/DirectSum/Decomposition.lean,Mathlib/Algebra/DirectSum/Internal.lean,Mathlib/Algebra/DirectSum/Ring.lean,Mathlib/Algebra/EuclideanDomain/Defs.lean,Mathlib/Algebra/Field/Defs.lean,Mathlib/Algebra/GCDMonoid/Div.lean,Mathlib/Algebra/GeomSum.lean,Mathlib/Algebra/GroupWithZero/Basic.lean,Mathlib/Algebra/GroupWithZero/Commute.lean,Mathlib/Algebra/GroupWithZero/Units/Basic.lean,Mathlib/Algebra/Homology/Additive.lean,Mathlib/Algebra/Homology/ComplexShape.lean,Mathlib/Algebra/Homology/Homology.lean,Mathlib/Algebra/Homology/Homotopy.lean,Mathlib/Algebra/Homology/HomotopyCategory.lean,Mathlib/Algebra/Homology/ImageToKernel.lean,Mathlib/Algebra/IndicatorFunction.lean,Mathlib/Algebra/LinearRecurrence.lean,Mathlib/Algebra/Module/BigOperators.lean,Mathlib/Algebra/Module/GradedModule.lean,Mathlib/Algebra/Module/LinearMap.lean,Mathlib/Algebra/Module/PointwisePi.lean,Mathlib/Algebra/Module/Submodule/Basic.lean,Mathlib/Algebra/Module/Submodule/Bilinear.lean,Mathlib/Algebra/Module/Submodule/Lattice.lean,Mathlib/Algebra/Module/Submodule/Pointwise.lean,Mathlib/Algebra/Module/Torsion.lean,Mathlib/Algebra/MonoidAlgebra/Basic.lean,Mathlib/Algebra/MonoidAlgebra/Degree.lean,Mathlib/Algebra/Order/Chebyshev.lean,Mathlib/Algebra/Order/Module.lean,Mathlib/Algebra/Order/Pointwise.lean,Mathlib/Algebra/Order/Rearrangement.lean,Mathlib/Algebra/Order/SMul.lean,Mathlib/Algebra/Order/UpperLower.lean,Mathlib/Algebra/Periodic.lean,Mathlib/Algebra/Polynomial/BigOperators.lean,Mathlib/Algebra/Polynomial/GroupRingAction.lean,Mathlib/Algebra/Star/BigOperators.lean,Mathlib/Algebra/Star/Pointwise.lean,Mathlib/Algebra/Star/Subalgebra.lean,Mathlib/Algebra/Support.lean,Mathlib/Algebra/TrivSqZeroExt.lean,Mathlib/Algebra/Tropical/BigOperators.lean,Mathlib/AlgebraicGeometry/PrimeSpectrum/Basic.lean,Mathlib/AlgebraicGeometry/PrimeSpectrum/Maximal.lean,Mathlib/AlgebraicGeometry/ProjectiveSpectrum/Topology.lean,Mathlib/AlgebraicTopology/AlternatingFaceMapComplex.lean,Mathlib/AlgebraicTopology/ExtraDegeneracy.lean,Mathlib/AlgebraicTopology/TopologicalSimplex.lean,Mathlib/Analysis/Analytic/Basic.lean,Mathlib/Analysis/Asymptotics/AsymptoticEquivalent.lean,Mathlib/Analysis/Asymptotics/Asymptotics.lean,Mathlib/Analysis/Asymptotics/SpecificAsymptotics.lean,Mathlib/Analysis/Asymptotics/SuperpolynomialDecay.lean,Mathlib/Analysis/Asymptotics/Theta.lean,Mathlib/Analysis/BoxIntegral/Box/Basic.lean,Mathlib/Analysis/BoxIntegral/Box/SubboxInduction.lean,Mathlib/Analysis/BoxIntegral/Partition/Additive.lean,Mathlib/Analysis/BoxIntegral/Partition/Basic.lean,Mathlib/Analysis/BoxIntegral/Partition/Filter.lean,Mathlib/Analysis/BoxIntegral/Partition/Split.lean,Mathlib/Analysis/BoxIntegral/Partition/SubboxInduction.lean,Mathlib/Analysis/BoxIntegral/Partition/Tagged.lean,Mathlib/Analysis/Calculus/ContDiffDef.lean,Mathlib/Analysis/Calculus/Deriv/Add.lean |
788 |
0 |
[] |
nobody |
409-8937 1 year ago |
430-76042 1 year ago |
0-0 0 seconds |
3757 |
thorimur author:thorimur |
feat: config options for `fail_if_no_progress` |
This PR creates config options for `fail_if_no_progress` that allow the user to tweak what exactly counts as "progress". This includes whether to use defeq or `BEq`, what transparency to use, and which parts of the goal and local context to check.
It also splits off the comparison functionality into `Mathlib.Lean.Meta.Compare`, which provides fully configurable comparison functions for common complex metaprogramming types not specific to `fail_if_no_progress`. These types are `Expr`, `LocalDecl`, `LocalContext`, `MetavarDecl`, `MVarId`, and `List MVarId`.
---
See [zulip](https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/progress.20on.20fail_if_no_progress) for a couple review questions.
Status update: this PR is now basically done, save for some extra tests which should probably be included.
[](https://gitpod.io/from-referrer/)
|
t-meta
merge-conflict
WIP
|
603/54 |
Mathlib.lean,Mathlib/Lean/Meta.lean,Mathlib/Lean/Meta/Compare.lean,Mathlib/Tactic/FailIfNoProgress.lean,test/fail_if_no_progress.lean |
5 |
38 |
['alexjbest', 'github-actions', 'joneugster', 'kim-em', 'thorimur'] |
nobody |
409-8936 1 year ago |
661-20122 1 year ago |
45-49113 45 days |
12353 |
thorimur author:thorimur |
feat: `conv%` |
This PR introduces `conv% e => tac`, along with `simp%`, `norm_num%`, and `push_neg%`, which are defined in terms of `conv%`.
It also introduces `conv%?` (and `simp%?`, `norm_num%?`, and `push_neg%?`) as shortcuts for `show_term ...`.
This is a relatively straightforward refactor of code already present in the implementation of `#conv`, and otherwise relies entirely on simple macros.
This PR also introduces some modifications to existing command syntax for `#conv`, `#simp`, and `#norm_num`:
* The syntax for `#conv` was `#conv tac => e`; however, this is inconsistent with the tactic syntax, and so this has been flipped to `#conv e => tac`. Likewise, `conv%` uses the same (new) syntax `conv% e => tac`.
* `#simp` and `#norm_num` separated their config and `only` syntax from the expression by an optional `=>` (for `#simp`) and an optional `:` (for `#norm_num`) (e.g. `#simp only [lem] => e`). These have both been replaced with an optional`on` (e.g. `#simp only [lem] on e`) which is also used for `simp%` and `norm_num%`.
Although `#whnf` is implemented in terms of `#conv`, this PR doesn't introduce `whnf%` in the same way, as that's probably better off being implemented directly instead of through `conv`.
---
WIP: needs tests.
[](https://gitpod.io/from-referrer/)
|
t-meta
merge-conflict
WIP
|
131/32 |
Mathlib/Tactic/Conv.lean,Mathlib/Tactic/NormNum/Core.lean,Mathlib/Tactic/PushNeg.lean,docs/Conv/Guide.lean |
4 |
0 |
[] |
nobody |
404-71646 1 year ago |
404-71646 1 year ago |
0-0 0 seconds |
7903 |
urkud author:urkud |
feat: define `UnboundedSpace` |
---
The new instances generate some timeouts, and I don't understand why.
[](https://gitpod.io/from-referrer/)
|
t-topology
merge-conflict
help-wanted
|
111/59 |
Mathlib/Analysis/BoxIntegral/Basic.lean,Mathlib/Analysis/Normed/Module/Basic.lean,Mathlib/Topology/Bornology/Basic.lean,Mathlib/Topology/Bornology/Constructions.lean,Mathlib/Topology/MetricSpace/Bounded.lean,Mathlib/Topology/MetricSpace/GromovHausdorffRealized.lean |
6 |
1 |
['github-actions'] |
nobody |
401-83315 1 year ago |
401-83315 1 year ago |
0-0 0 seconds |
14994 |
kim-em author:kim-em |
profiling: skipKernelTC |
|
merge-conflict |
2/1 |
lakefile.lean |
1 |
3 |
['github-actions', 'kim-em', 'leanprover-bot'] |
nobody |
400-29059 1 year ago |
400-29059 1 year ago |
0-0 0 seconds |
15400 |
grunweg author:grunweg |
feat: "confusing variables" linter |
This linter flags `variable` commands which both update an existing binder annotation and declare new variables: these can yield confusing or misleading error messages (see leanprover/lean4#2789).
Instead, these should be split in several `variable` statements.
----------
Help fixing these errors is welcome!
Currently, the linter only catches *some* cases, when the updated binder is from a previous scope.
To make it catch all cases, the linter could insert a `section` before the `variable` command and use that scope instead.
See [zulip](https://leanprover.zulipchat.com/#narrow/stream/113488-general/topic/Get.20scope.20*before*.20some.20syntax.20is.20evaluated) [discussions](https://leanprover.zulipchat.com/#narrow/stream/113488-general/topic/Determining.20variable.20binders.20from.20syntax).
---
[](https://gitpod.io/from-referrer/)
|
t-linter
merge-conflict
WIP
|
292/47 |
Cache/Requests.lean,Mathlib/Analysis/NormedSpace/OperatorNorm/Prod.lean,Mathlib/Dynamics/Ergodic/Ergodic.lean,Mathlib/FieldTheory/AbelRuffini.lean,Mathlib/FieldTheory/Adjoin.lean,Mathlib/FieldTheory/IntermediateField.lean,Mathlib/FieldTheory/KummerExtension.lean,Mathlib/FieldTheory/Minpoly/MinpolyDiv.lean,Mathlib/FieldTheory/Normal.lean,Mathlib/FieldTheory/PurelyInseparable.lean,Mathlib/Geometry/Manifold/BumpFunction.lean,Mathlib/Geometry/Manifold/ChartedSpace.lean,Mathlib/Geometry/Manifold/ContMDiff/Basic.lean,Mathlib/Geometry/Manifold/PartitionOfUnity.lean,Mathlib/Geometry/Manifold/VectorBundle/Basic.lean,Mathlib/Geometry/Manifold/VectorBundle/Tangent.lean,Mathlib/LinearAlgebra/CliffordAlgebra/Basic.lean,Mathlib/Tactic/Linter/Lint.lean,Mathlib/Tactic/ToAdditive/Frontend.lean,Mathlib/Topology/FiberBundle/Basic.lean,Mathlib/Topology/FiberBundle/Trivialization.lean,test/Lint.lean |
22 |
1 |
['github-actions'] |
nobody |
396-76409 1 year ago |
402-27031 1 year ago |
0-0 0 seconds |
14654 |
grunweg author:grunweg |
feat(runLinter): allow only running certain linters |
This adds a script `run_linter`, which is a fork of batteries' `runLinter` with extra features:
- rewrite as a CLI app, so --help messages etc. come for free
- add a `--list` option, which prints the list of linters it was about to run, and exists
- add `--select`, `--ignore` and `--only` options which ensure certain linters are always run, never resp. that only a certain list of linters are run. (`add` takes priority over `exclude` or `only`.)
- add an `update_only_remove` flag which only runs linters mentioned in the `nolints` file: this only removes entries (by design), but is often much faster.
- renamed to `run_linter`: actually, per the [zulip discussion](https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/Naming.20convention/near/450896930), this should be `run-linter` --- and one could as well use the opportunity to rename this to e.g. `env-linter`. Asked [here](https://leanprover.zulipchat.com/#narrow/stream/270676-lean4/topic/Configuring.2Fmodernizing.20runLinter).
Intended use cases
1. Run `update_only_remove` when updating the nolints file. In fact, it is so fast that it could even run during regular CI, after the normal `lint` step...
2. Run the mathlib linters locally. The simpNF linters are slow enough (for a reason, but still) that doing so is currently annoying. On my notebook, they can easily take half an hour, during which my notebook is otherwise hardly usable.
3. You're developing a new linter and only want to run *that* one (as there was no change about the other ones).
Probably, the nicest result would be this PR landing in batteries (perhaps in pieces) instead of here.
---
Two CLI warts I'm unhappy about.
- how can I have flag names with a hyphen? Currently, I have to write `--print_linters`, which is less pretty.
- many options take an `Array String`: how can I pass this to the executable? This is not obvious to me...
[](https://gitpod.io/from-referrer/)
|
t-linter
RFC
merge-conflict
|
320/146 |
Mathlib/Analysis/LocallyConvex/Bounded.lean,Mathlib/Analysis/Oscillation.lean,Mathlib/Geometry/Manifold/LocalInvariantProperties.lean,Mathlib/MeasureTheory/Measure/EverywherePos.lean,Mathlib/SetTheory/Ordinal/Topology.lean,Mathlib/Topology/Algebra/Group/Basic.lean,Mathlib/Topology/Algebra/Module/Basic.lean,Mathlib/Topology/Algebra/Monoid.lean,Mathlib/Topology/Bases.lean,Mathlib/Topology/Basic.lean,Mathlib/Topology/Category/TopCat/Basic.lean,Mathlib/Topology/Clopen.lean,Mathlib/Topology/CompactOpen.lean,Mathlib/Topology/Compactness/LocallyCompact.lean,Mathlib/Topology/Constructions.lean,Mathlib/Topology/ContinuousOn.lean,Mathlib/Topology/DenseEmbedding.lean,Mathlib/Topology/Gluing.lean,Mathlib/Topology/Homeomorph.lean,Mathlib/Topology/IndicatorConstPointwise.lean,Mathlib/Topology/Inseparable.lean,Mathlib/Topology/Irreducible.lean,Mathlib/Topology/IsLocalHomeomorph.lean,Mathlib/Topology/LocalAtTarget.lean,Mathlib/Topology/Maps/Basic.lean,Mathlib/Topology/MetricSpace/Isometry.lean,Mathlib/Topology/NoetherianSpace.lean,Mathlib/Topology/Order.lean,Mathlib/Topology/Order/LowerUpperTopology.lean,Mathlib/Topology/Partial.lean,Mathlib/Topology/PartialHomeomorph.lean,Mathlib/Topology/PartitionOfUnity.lean,Mathlib/Topology/QuasiSeparated.lean,Mathlib/Topology/Separation.lean,Mathlib/Topology/TietzeExtension.lean,Mathlib/Topology/UniformSpace/Ascoli.lean,Mathlib/Topology/UniformSpace/Basic.lean,Mathlib/Topology/UniformSpace/Cauchy.lean,Mathlib/Topology/UniformSpace/CompactConvergence.lean,Mathlib/Topology/UniformSpace/Completion.lean,Mathlib/Topology/UniformSpace/Equicontinuity.lean,Mathlib/Topology/UniformSpace/Matrix.lean,Mathlib/Topology/UniformSpace/Pi.lean,Mathlib/Topology/UnitInterval.lean,Mathlib/Topology/UrysohnsBounded.lean,Mathlib/Topology/UrysohnsLemma.lean,Mathlib/Topology/VectorBundle/Basic.lean,lakefile.lean,scripts/run_linter.lean |
49 |
5 |
['github-actions', 'grunweg', 'rosborn'] |
nobody |
396-53259 1 year ago |
396-53259 1 year ago |
13-61906 13 days |
15679 |
adomani author:adomani |
test: refactor in CI |
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict
WIP
|
213/5 |
.github/workflows/bors.yml,.github/workflows/build.yml,.github/workflows/build.yml.in,.github/workflows/build_fork.yml,Mathlib.lean,Mathlib/Algebra/Homology/HomotopyCategory/SingleFunctors.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Affine.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Order.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Unique.lean,Mathlib/Analysis/Convex/Combination.lean,Mathlib/Analysis/Convex/Segment.lean,Mathlib/CategoryTheory/Bicategory/Adjunction.lean,Mathlib/CategoryTheory/Monoidal/Braided/Basic.lean,Mathlib/CategoryTheory/Monoidal/Center.lean,Mathlib/GroupTheory/Coxeter/Matrix.lean,Mathlib/Order/Filter/Cocardinal.lean,Mathlib/Order/UpperLower/Basic.lean,Mathlib/TestRefactor.lean,Refactor/Main.lean,lakefile.lean,lean-toolchain |
21 |
1 |
['github-actions'] |
nobody |
396-52491 1 year ago |
396-52491 1 year ago |
0-8 8 seconds |
10629 |
madvorak author:madvorak |
feat: List.cons_sublist_append_iff_right |
---
[](https://gitpod.io/from-referrer/)
|
t-data
merge-conflict
|
11/0 |
Mathlib/Data/List/Basic.lean |
1 |
1 |
['eric-wieser'] |
nobody |
395-2482 1 year ago |
395-2482 1 year ago |
53-73442 53 days |
9973 |
Ruben-VandeVelde author:Ruben-VandeVelde |
feat: polynomials formed by lists |
From https://github.com/leanprover-community/mathlib/pull/15476
---
[](https://gitpod.io/from-referrer/)
|
t-data
merge-conflict
please-adopt
|
311/0 |
Mathlib.lean,Mathlib/Data/Polynomial/OfList.lean |
2 |
0 |
[] |
nobody |
395-2015 1 year ago |
395-2015 1 year ago |
0-0 0 seconds |
12926 |
joelriou author:joelriou |
feat(CategoryTheory): the monoidal category structure induced by a monoidal functor |
In this PR, given a monoidal functor `F : MonoidalFunctor C D`, we define a monoidal category structure on the category `InducedCategory D F.obj`, which has the "same" objects as `C`, but the morphisms between `X` and `Y` identify to `F.obj X ⟶ F.obj Y`.
---
[](https://gitpod.io/from-referrer/)
|
t-category-theory
merge-conflict
WIP
|
105/0 |
Mathlib.lean,Mathlib/CategoryTheory/Monoidal/Induced.lean |
2 |
3 |
['eric-wieser', 'github-actions', 'joelriou'] |
nobody |
395-414 1 year ago |
395-414 1 year ago |
0-0 0 seconds |
12869 |
adomani author:adomani |
feat: linter and script for `theorem` vs `lemma` |
This PR contains a linter for flagging doc-string-less `theorem`s, as well as a bash script that, once the linter ran on Mathlib, automatically replaces every linter-offending `theorem` by `lemma`.
---
[](https://gitpod.io/from-referrer/)
|
t-linter
merge-conflict
awaiting-author
|
106/0 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter/ThmLemma.lean,scripts/thmLemma.sh |
4 |
13 |
['adomani', 'github-actions', 'grunweg', 'joneugster'] |
nobody |
394-73578 1 year ago |
394-73578 1 year ago |
0-0 0 seconds |
14308 |
grhkm21 author:grhkm21 |
feat(Algebra/Category): Direct construction of colimits in algebraic categories |
(Below I only write about colimits since that's what I'm familiar with after working on it the last few days, but maybe it's the same for other categorical constructions)
**Main feature:** Construct colimits in `AddCommGrp`/`ModuleCat`/`FGModuleCat`(/...) directly as coequalizer (i.e. cokernel i.e. quotient) of two maps, allowing one to say $\coprod_j M_j \cong *$
Currently, if you look at how colimits are constructed for [AddCommGrp](https://github.com/leanprover-community/mathlib4/blob/master/Mathlib/Algebra/Category/Grp/Colimits.lean#L69-L92), you see this massive block of code of all relations generating the quotient relation, but that's kind of bad, you can't say anything concretely about it.
Also as noted in the TODOs of a few files:
```
TODO:
In fact, in `ModuleCat R` there is a much nicer model of colimits as quotients
of finitely supported functions, and we really should implement this as well.
```
I wrote it down [here](https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/Braided.20left.20rigid.20categories.20are.20right.20rigid/near/447490672), and **have formalised it** in a small file already [here](https://gist.github.com/grhkm21/5b2d938753c0ce0900d21c93a39e3b7d#file-addcommgrpcolimits-lean-L162-L163) (I also have a `ModuleCat` version, and proving existence of colimits in `FGModuleCat` from it).
Usually I will try to merge the file into Mathlib directly (preferably in one sitting), but I have been trying for a while now and been struggling. One issue is I am struggling to understand universes, which I asked [here](https://leanprover.zulipchat.com/#narrow/stream/113489-new-members/topic/Universe.20constraints!/near/448049266) along with many other places. A more concrete issue is that
- [ ] FGModuleCat (and `FullSubcategory` in general) requires morphism and objects to be on the same universe, whereas generally `Category.{v, u}` don't.
So that seems to limit what I can express, and maybe I have to fix it first.
Here are a few more TODOs just so I don't forget, probably done before the one above:
- [ ] Generalise `cokernelIsoQuotient` to other categories.
- [ ] Also prove `coproductIsoDirectSum`
- [ ] Also prove coequalizer (f + h) (g + h) ~ coequalizer f g ~ cokernel (f - g) 0
- [ ] Fix typo `FGModuleCatCat`
If anyone is familiar with universe stuff and can answer my many questions that'll be great too. I need help understanding just [these five lines](https://github.com/leanprover-community/mathlib4/blob/master/Mathlib/Algebra/Category/Grp/Colimits.lean#L267-L271) |
t-algebra
merge-conflict
WIP
label:t-algebra$ |
10/3 |
Mathlib/Algebra/DirectSum/Module.lean,Mathlib/LinearAlgebra/FreeModule/Basic.lean |
2 |
1 |
['github-actions'] |
nobody |
393-85599 1 year ago |
393-85599 1 year ago |
0-0 0 seconds |
13010 |
ADedecker author:ADedecker |
feat: relax universe constraint in stoneCechExtend |
---
[](https://gitpod.io/from-referrer/)
|
t-topology
merge-conflict
|
33/3 |
Mathlib/Topology/StoneCech.lean |
1 |
2 |
['ADedecker', 'erdOne'] |
nobody |
393-85396 1 year ago |
393-85396 1 year ago |
0-0 0 seconds |
12411 |
adomani author:adomani |
feat: more linting of cdots |
---
[](https://gitpod.io/from-referrer/)
|
t-linter
merge-conflict
|
953/617 |
Archive/Wiedijk100Theorems/CubingACube.lean,Mathlib.lean,Mathlib/Algebra/Category/GroupCat/Colimits.lean,Mathlib/Algebra/Homology/Exact.lean,Mathlib/Algebra/Homology/LocalCohomology.lean,Mathlib/Algebra/Lie/Nilpotent.lean,Mathlib/Algebra/Module/PID.lean,Mathlib/Algebra/Module/Submodule/Bilinear.lean,Mathlib/Algebra/Module/Torsion.lean,Mathlib/Algebra/MonoidAlgebra/Basic.lean,Mathlib/Algebra/Order/Archimedean.lean,Mathlib/AlgebraicGeometry/StructureSheaf.lean,Mathlib/Analysis/Analytic/Composition.lean,Mathlib/Analysis/Calculus/Deriv/Slope.lean,Mathlib/Analysis/Calculus/InverseFunctionTheorem/ApproximatesLinearOn.lean,Mathlib/Analysis/Calculus/LocalExtr/Basic.lean,Mathlib/Analysis/Calculus/TangentCone.lean,Mathlib/Analysis/InnerProductSpace/Basic.lean,Mathlib/Analysis/InnerProductSpace/Projection.lean,Mathlib/Analysis/MeanInequalitiesPow.lean,Mathlib/Analysis/Normed/Group/ControlledClosure.lean,Mathlib/Analysis/Normed/Group/Pointwise.lean,Mathlib/Analysis/NormedSpace/FiniteDimension.lean,Mathlib/Analysis/NormedSpace/HahnBanach/Separation.lean,Mathlib/Analysis/NormedSpace/Multilinear/Basic.lean,Mathlib/Analysis/NormedSpace/Star/Basic.lean,Mathlib/Analysis/NormedSpace/Star/Multiplier.lean,Mathlib/Analysis/NormedSpace/lpSpace.lean,Mathlib/Analysis/PSeries.lean,Mathlib/Analysis/RCLike/Basic.lean,Mathlib/Analysis/SpecialFunctions/Complex/Arg.lean,Mathlib/Analysis/SpecialFunctions/Log/Base.lean,Mathlib/Analysis/SpecialFunctions/Log/Monotone.lean,Mathlib/Analysis/SpecialFunctions/Pow/NNReal.lean,Mathlib/Analysis/SpecialFunctions/Pow/Real.lean,Mathlib/Analysis/SpecificLimits/Normed.lean,Mathlib/CategoryTheory/Abelian/Basic.lean,Mathlib/CategoryTheory/Action.lean,Mathlib/CategoryTheory/Bicategory/NaturalTransformation.lean,Mathlib/CategoryTheory/Category/Cat/Limit.lean,Mathlib/CategoryTheory/Category/PartialFun.lean,Mathlib/CategoryTheory/Category/TwoP.lean,Mathlib/CategoryTheory/Closed/Cartesian.lean,Mathlib/CategoryTheory/Functor/Flat.lean,Mathlib/CategoryTheory/Galois/GaloisObjects.lean,Mathlib/CategoryTheory/Limits/Over.lean,Mathlib/CategoryTheory/Limits/VanKampen.lean,Mathlib/CategoryTheory/Localization/Predicate.lean,Mathlib/CategoryTheory/Monad/Coequalizer.lean,Mathlib/CategoryTheory/Monad/Monadicity.lean,Mathlib/CategoryTheory/Pi/Basic.lean,Mathlib/CategoryTheory/Sites/DenseSubsite.lean,Mathlib/CategoryTheory/Sites/InducedTopology.lean,Mathlib/CategoryTheory/Subobject/Lattice.lean,Mathlib/Combinatorics/Additive/PluenneckeRuzsa.lean,Mathlib/Combinatorics/HalesJewett.lean,Mathlib/Combinatorics/SimpleGraph/Regularity/Chunk.lean,Mathlib/Computability/Reduce.lean,Mathlib/Data/Holor.lean,Mathlib/Data/Nat/Multiplicity.lean,Mathlib/Data/Nat/Pairing.lean,Mathlib/Data/Real/Cardinality.lean,Mathlib/Data/Real/Hyperreal.lean,Mathlib/Data/Real/Irrational.lean,Mathlib/Data/Set/Card.lean,Mathlib/Dynamics/Circle/RotationNumber/TranslationNumber.lean,Mathlib/FieldTheory/Finite/Polynomial.lean,Mathlib/FieldTheory/Minpoly/IsIntegrallyClosed.lean,Mathlib/FieldTheory/PerfectClosure.lean,Mathlib/FieldTheory/RatFunc.lean,Mathlib/Geometry/RingedSpace/OpenImmersion.lean,Mathlib/Geometry/RingedSpace/PresheafedSpace/Gluing.lean,Mathlib/GroupTheory/GroupAction/Quotient.lean,Mathlib/GroupTheory/Nilpotent.lean,Mathlib/GroupTheory/Perm/Cycle/Factors.lean,Mathlib/GroupTheory/Perm/Finite.lean,Mathlib/GroupTheory/SpecificGroups/Quaternion.lean,Mathlib/GroupTheory/Sylow.lean,Mathlib/LinearAlgebra/Dimension/RankNullity.lean,Mathlib/LinearAlgebra/Dual.lean,Mathlib/LinearAlgebra/LinearIndependent.lean,Mathlib/LinearAlgebra/LinearPMap.lean,Mathlib/LinearAlgebra/Matrix/Charpoly/Coeff.lean,Mathlib/LinearAlgebra/Prod.lean,Mathlib/LinearAlgebra/QuadraticForm/Complex.lean,Mathlib/LinearAlgebra/Reflection.lean,Mathlib/MeasureTheory/Constructions/Pi.lean,Mathlib/MeasureTheory/Covering/VitaliFamily.lean,Mathlib/MeasureTheory/Measure/Haar/Basic.lean,Mathlib/MeasureTheory/Measure/MeasureSpace.lean,Mathlib/MeasureTheory/Measure/Typeclasses.lean,Mathlib/MeasureTheory/OuterMeasure/Basic.lean,Mathlib/ModelTheory/Skolem.lean,Mathlib/NumberTheory/Dioph.lean,Mathlib/NumberTheory/LegendreSymbol/Basic.lean,Mathlib/NumberTheory/Padics/Hensel.lean,Mathlib/NumberTheory/Padics/PadicNumbers.lean,Mathlib/NumberTheory/Padics/RingHoms.lean,Mathlib/NumberTheory/RamificationInertia.lean,Mathlib/RingTheory/AdjoinRoot.lean |
147 |
2 |
['adomani', 'leanprover-bot'] |
nobody |
393-85259 1 year ago |
393-85259 1 year ago |
0-0 0 seconds |
12279 |
casavaca author:casavaca |
WIP: feat: Holder's inequality n-ary |
---
- [x] depends on #12291
[](https://gitpod.io/from-referrer/)
|
t-analysis
merge-conflict
WIP
|
129/0 |
Mathlib/Analysis/MeanInequalities.lean,Mathlib/Analysis/SpecialFunctions/Pow/Real.lean |
2 |
13 |
['github-actions'] |
nobody |
393-85244 1 year ago |
393-85244 1 year ago |
0-0 0 seconds |
12093 |
ADedecker author:ADedecker |
feat: tweak the definition of semicontinuity to behave better in nonlinear orders |
Summary of the changes:
- change definitions to make [lowerSemicontinuous_iff_isClosed_preimage](https://leanprover-community.github.io/mathlib4_docs/Mathlib/Topology/Semicontinuous.html#lowerSemicontinuous_iff_isClosed_preimage) true without assuming `LinearOrder`, so that semicontinuity corresponds to continuity for lower/upper order topology on the codomain. See discussion on [Zulip](https://leanprover.zulipchat.com/#narrow/stream/116395-maths/topic/Semicontinuity.20definition.20for.20non-linear.20orders/near/432898278)
- add new `iff` lemmas for unfolding the definition
- add `iff` lemmas with the old definition in the linearly ordered case
- some basic lemmas need to be changed in an easy way
- minimize assumptions for continuity => semicontinuity
- prove the semicontinuity criterion for indicators using "preimage of Ici/Iic" instead of a direct proof, because the proof is more natural (especially because we have no `filter_upwards` for `Frequently`)
- in the rest of the file (which is about linear orders anyway), we don't touch the statements and just rewrite to the old definition. Some of these could be generalized, but we keep that for a later PR.
---
[](https://gitpod.io/from-referrer/)
|
t-topology
merge-conflict
WIP
|
274/130 |
Mathlib/Analysis/BoundedVariation.lean,Mathlib/MeasureTheory/Integral/FundThmCalculus.lean,Mathlib/Order/Filter/Basic.lean,Mathlib/Topology/Semicontinuous.lean |
4 |
0 |
[] |
nobody |
393-85206 1 year ago |
393-85206 1 year ago |
0-0 0 seconds |
11519 |
thorimur author:thorimur |
feat: `syntax_rules` |
---
Experimental. WIP.
[](https://gitpod.io/from-referrer/)
|
t-meta
merge-conflict
|
485/0 |
Mathlib.lean,Mathlib/Command/SyntaxRules.lean,Mathlib/Command/SyntaxRules/Attr.lean,Mathlib/Command/SyntaxRules/Elab.lean,Mathlib/Command/SyntaxRules/Header.lean,Mathlib/Command/SyntaxRules/Util.lean,scripts/noshake.json |
7 |
0 |
[] |
nobody |
393-85182 1 year ago |
393-85182 1 year ago |
0-0 0 seconds |
11393 |
mcdoll author:mcdoll |
feat(Analysis/Distribution/SchwartzSpace): The Heine-Borel property |
---
[](https://gitpod.io/from-referrer/)
|
t-analysis
merge-conflict
WIP
|
688/3 |
Mathlib.lean,Mathlib/Analysis/Distribution/SchwartzSpace.lean,Mathlib/Topology/Constructions.lean,Mathlib/Topology/UniformSpace/Ascoli.lean,Mathlib/Topology/UniformSpace/Pi.lean,Mathlib/Topology/UniformSpace/UniformConvergenceTopology.lean |
6 |
0 |
[] |
nobody |
393-85172 1 year ago |
393-85172 1 year ago |
0-0 0 seconds |
9444 |
erdOne author:erdOne |
feat: Various instances regarding `𝓞 K`. |
---
[](https://gitpod.io/from-referrer/)
|
t-number-theory
merge-conflict
help-wanted
|
27/0 |
Mathlib/NumberTheory/NumberField/Basic.lean,Mathlib/RingTheory/IntegralClosure.lean |
2 |
9 |
['erdOne', 'leanprover-bot', 'mattrobball', 'riccardobrasca', 'xroblot'] |
nobody |
393-85091 1 year ago |
393-85091 1 year ago |
0-0 0 seconds |
8931 |
hmonroe author:hmonroe |
feat(Computable): define P, NP, and NP-complete |
Revised to focus on languages that are binary strings, given the issue of non-acceptable encodings of unspecified Types
---
[](https://gitpod.io/from-referrer/)
|
t-computability
merge-conflict
awaiting-author
|
381/5 |
Mathlib.lean,Mathlib/Computability/Complexity copy.lean,Mathlib/Computability/Complexity.lean,Mathlib/Computability/Encoding.lean,Mathlib/Computability/TMComputable.lean,Mathlib/Computability/TuringMachine.lean,Mathlib/Computability/halting example.lean,docs/references.bib |
8 |
3 |
['fpvandoorn', 'github-actions', 'hmonroe'] |
nobody |
393-85056 1 year ago |
393-85056 1 year ago |
5-62479 5 days |
10641 |
newell author:newell |
feat(Topology/MetricSpace/WellSpaced): Define sets that are *well-spaced*. |
Create a new file `Mathlib.Topology.MetricSpace.WellSpaced` that contains definitions of sets which are in some sense *well-spaced*.
Some examples are Delone and Meyer sets, which find applications in Quasicrystals and Coding Theory, among others.
---
[](https://gitpod.io/from-referrer/)
|
t-topology
merge-conflict
|
1073/14 |
Mathlib.lean,Mathlib/Analysis/LocallyConvex/WithSeminorms.lean,Mathlib/Topology/EMetricSpace/Basic.lean,Mathlib/Topology/GMetric/Basic.lean,Mathlib/Topology/GMetric/GInfSep.lean,Mathlib/Topology/GMetric/WellSpaced.lean,Mathlib/Topology/GPseudoMetric/Basic.lean,Mathlib/Topology/MetricSpace/WellSpaced.lean |
8 |
1 |
['edegeltje'] |
nobody |
393-85024 1 year ago |
393-85024 1 year ago |
0-0 0 seconds |
10428 |
dwrensha author:dwrensha |
feat: add simp_digits tactic |
With the introduction of the simprocs `reduceLE`, `reduceMod`, `reduceDiv` etc. in Lean v4.6.0, now `simp`
can fully normalize typical `Nat.digits` calls that have concrete arguments. The situation is still a bit delicate
however, as we want to avoid invoking kernel reduction on `Nat.digits`, because the `Acc`-based ("well founded")
recursion in `digitsAux` can get bogged down.
This PR introduces a new tactic `simp_digits` tactic that contains only the simp lemmas and simprocs needed
to reduce `Nat.digits`. This allows proofs involving `Nat.digits` to be cleanly factored into two steps:
1. reduce `Nat.digits` via `simp_digits`,
2. do things that require kernel reduction such as `simp_arith`, `decide`, or `rfl`.
---
[](https://gitpod.io/from-referrer/)
|
t-meta
merge-conflict
|
6/124 |
Archive/Imo/Imo1960Q1.lean,Archive/Imo/Imo1962Q1.lean,Mathlib/Data/Nat/Digits.lean |
3 |
2 |
['dwrensha'] |
nobody |
393-84878 1 year ago |
393-84878 1 year ago |
0-0 0 seconds |
8608 |
eric-wieser author:eric-wieser |
feat: multiplicativize `AddTorsor` |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
WIP
label:t-algebra$ |
268/199 |
Mathlib/Algebra/AddTorsor.lean,Mathlib/Algebra/Group/Defs.lean,Mathlib/Data/Set/Pointwise/SMul.lean,Mathlib/Tactic/ToAdditive.lean |
4 |
0 |
[] |
nobody |
393-84701 1 year ago |
393-84701 1 year ago |
0-0 0 seconds |
6603 |
tydeu author:tydeu |
feat: automatically try `cache get` before build |
---
A quick proof-of-concept. With this, `lake build` will always try `cache get` before building mathlib.
[](https://gitpod.io/from-referrer/)
|
CI
merge-conflict
WIP
|
29/0 |
lakefile.lean |
1 |
3 |
['kim-em', 'tydeu'] |
nobody |
393-84643 1 year ago |
393-84643 1 year ago |
11-1960 11 days |
6058 |
apurvnakade author:apurvnakade |
feat: duality theory for cone programs |
This PR tracks the development of duality theory for cone programs.
[Reference](https://ti.inf.ethz.ch/ew/courses/ApproxSDP09/notes/conelp.pdf)
---
[](https://gitpod.io/from-referrer/)
- [x] depends on: #6059
- [ ] define direct sum of cones
- [ ] weak duality
- [ ] regular duality
- [ ] slater condition
- [ ] strong duality |
t-analysis
merge-conflict
WIP
|
159/0 |
Mathlib.lean,Mathlib/Analysis/Convex/Cone/ConeLinearProgram.lean |
2 |
1 |
['leanprover-community-mathlib4-bot'] |
nobody |
393-84588 1 year ago |
393-84588 1 year ago |
0-0 0 seconds |
6449 |
ADedecker author:ADedecker |
feat: functions with finite fibers |
---
This has been discussed before on [Zulip](https://leanprover.zulipchat.com/#narrow/stream/217875-Is-there-code-for-X.3F/topic/.E2.9C.94.20Cofinite.20maps.3F) and it came up again while working with @kkytola's student. As explained in the docstring, we could absolutely just use `Tendsto f cofinite cofinite` all the time, but (1) we lack some API for it (2) the API is nicer to setup if we have a separate def (e.g for dot notation) and (3) mentioning filters for such a simple concept is really not beginner-friendly.
I'm not sure at all about the name.
[](https://gitpod.io/from-referrer/)
|
t-topology
merge-conflict
awaiting-author
|
203/0 |
Mathlib.lean,Mathlib/Logic/Function/HasFiniteFibers.lean,Mathlib/Order/Filter/Basic.lean,Mathlib/Order/Filter/Cofinite.lean |
4 |
14 |
['ADedecker', 'YaelDillies', 'alexjbest', 'kkytola'] |
nobody |
393-84582 1 year ago |
393-84582 1 year ago |
6-70040 6 days |
8100 |
digama0 author:digama0 |
feat: add support for other types in norm_num |
---
[](https://gitpod.io/from-referrer/)
|
t-meta
merge-conflict
|
177/12 |
Mathlib/Tactic/NormNum/Basic.lean,Mathlib/Tactic/NormNum/Eq.lean,Mathlib/Tactic/NormNum/Ineq.lean,Mathlib/Tactic/NormNum/Pow.lean,Mathlib/Tactic/NormNum/Result.lean,Mathlib/Tactic/NormNum/Structural.lean,test/norm_num.lean |
7 |
4 |
['dwrensha'] |
nobody |
393-84450 1 year ago |
393-84450 1 year ago |
0-0 0 seconds |
7739 |
mcdoll author:mcdoll |
feat(LinearAlgebra/LinearPMap): difference of inverses |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
WIP
label:t-algebra$ |
126/7 |
Mathlib/LinearAlgebra/LinearPMap.lean,lean-toolchain |
2 |
2 |
['digama0', 'eric-wieser'] |
nobody |
393-84422 1 year ago |
393-84422 1 year ago |
0-0 0 seconds |
15585 |
FR-vdash-bot author:FR-vdash-bot |
test make `HasQuotient.quotient'` reducible |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
label:t-algebra$ |
8/1 |
Mathlib/Algebra/Quotient.lean,Mathlib/GroupTheory/Coset.lean |
2 |
1 |
['github-actions'] |
nobody |
392-30458 1 year ago |
392-30458 1 year ago |
0-0 0 seconds |
15586 |
FR-vdash-bot author:FR-vdash-bot |
test make `HasQuotient` out put a `setoid` |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
label:t-algebra$ |
22/36 |
Mathlib/Algebra/Lie/CartanExists.lean,Mathlib/Algebra/Lie/Quotient.lean,Mathlib/Algebra/Lie/Weights/Basic.lean,Mathlib/Algebra/Quotient.lean,Mathlib/Analysis/Normed/Group/AddCircle.lean,Mathlib/GroupTheory/Commensurable.lean,Mathlib/GroupTheory/Coset.lean,Mathlib/GroupTheory/CosetCover.lean,Mathlib/GroupTheory/GroupAction/Quotient.lean,Mathlib/GroupTheory/Nilpotent.lean,Mathlib/GroupTheory/QuotientGroup.lean,Mathlib/LinearAlgebra/Quotient.lean,Mathlib/RingTheory/Ideal/Quotient.lean,Mathlib/Topology/Algebra/UniformRing.lean |
14 |
5 |
['FR-vdash-bot', 'github-actions', 'leanprover-bot'] |
nobody |
392-30458 1 year ago |
392-30458 1 year ago |
0-0 0 seconds |
13791 |
digama0 author:digama0 |
refactor: Primrec and Partrec |
General cleanup of the `Primrec` and `Partrec` files, to better adjust to lean 4 things. The main user-visible change is that `Primrec₂` is no longer a `def` but an `abbrev`, because it was causing inference issues in lean 4. I also removed all the nonterminal `simp`s in `PartrecCode.lean`.
---
[](https://gitpod.io/from-referrer/)
|
tech debt
t-computability
merge-conflict
|
585/778 |
Mathlib/Computability/Ackermann.lean,Mathlib/Computability/Halting.lean,Mathlib/Computability/Partrec.lean,Mathlib/Computability/PartrecCode.lean,Mathlib/Computability/Primrec.lean |
5 |
2 |
['github-actions', 'grunweg'] |
nobody |
390-51727 1 year ago |
430-76042 1 year ago |
1-84718 1 day |
11964 |
adamtopaz author:adamtopaz |
feat: The functor of points of a scheme |
We construct the functor of points functor, and prove that it's full and faithful.
---
- [ ] depends on: #11947
[](https://gitpod.io/from-referrer/)
|
t-algebraic-geometry
t-category-theory
merge-conflict
|
210/0 |
Mathlib.lean,Mathlib/AlgebraicGeometry/FunctorOfPoints.lean,Mathlib/AlgebraicGeometry/OpenImmersion.lean |
3 |
4 |
['github-actions', 'grunweg', 'leanprover-community-mathlib4-bot'] |
nobody |
390-51586 1 year ago |
430-76042 1 year ago |
0-1223 20 minutes |
12418 |
rosborn author:rosborn |
style: replace preimage_val with ↓∩ notation |
---
This is a rough draft of what the new `↓∩` notation would look like within mathlib. I believe this is an improvement in clarity and would like to have `↓∩` as a standard notation (along with `''`, `⁻¹'`, `↑`, etc...). As `↓∩` is specialized for `Set`s, I have only changed `preimage_val` when the left-hand side of `↓∩` is a `Set`.
The introduction of the `↓∩` notation to Data.Set.Image is temporary as it isn't possible to import Data.Set.Subset directly. If we want `↓∩` unscoped, where would be the best place to define it? An option is Data.Set.Defs, but the notation cannot be defined without additional imports as the file does not import `notation3`.
[](https://gitpod.io/from-referrer/)
|
merge-conflict |
56/61 |
Mathlib/Analysis/InnerProductSpace/Projection.lean,Mathlib/Data/Set/Function.lean,Mathlib/Data/Set/Image.lean,Mathlib/Data/Set/Subset.lean,Mathlib/MeasureTheory/Constructions/Polish.lean,Mathlib/MeasureTheory/MeasurableSpace/Basic.lean,Mathlib/MeasureTheory/Measure/Restrict.lean,Mathlib/Order/UpperLower/Basic.lean,Mathlib/Topology/Bases.lean,Mathlib/Topology/Clopen.lean,Mathlib/Topology/Connected/Basic.lean,Mathlib/Topology/Connected/PathConnected.lean,Mathlib/Topology/Constructions.lean,Mathlib/Topology/ContinuousOn.lean,Mathlib/Topology/LocalAtTarget.lean,Mathlib/Topology/LocallyConstant/Basic.lean,Mathlib/Topology/Separation.lean,Mathlib/Topology/Sober.lean |
18 |
3 |
['grunweg', 'rosborn'] |
nobody |
390-51485 1 year ago |
430-76042 1 year ago |
29-14218 29 days |
9978 |
FR-vdash-bot author:FR-vdash-bot |
chore(FieldTheory/KummerExtension): move some lemmas earlier |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
awaiting-author
label:t-algebra$ |
197/177 |
Mathlib.lean,Mathlib/Data/Polynomial/FieldDivision.lean,Mathlib/FieldTheory/KummerExtension.lean,Mathlib/RingTheory/AdjoinRoot.lean,Mathlib/RingTheory/Polynomial/Irreducible.lean |
5 |
5 |
['alreadydone', 'grunweg', 'riccardobrasca'] |
nobody |
390-51277 1 year ago |
390-51277 1 year ago |
8-83342 8 days |
12429 |
adomani author:adomani |
feat: toND -- auto-generating natDegree |
This is an experiment to automatically translate theorems about `degree` to theorems about `natDegree`.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
RFC
t-meta
merge-conflict
awaiting-author
label:t-algebra$ |
167/132 |
Mathlib.lean,Mathlib/Algebra/Polynomial/Degree/Definitions.lean,Mathlib/Algebra/Polynomial/Degree/Lemmas.lean,Mathlib/Algebra/Polynomial/EraseLead.lean,Mathlib/Algebra/Polynomial/HasseDeriv.lean,Mathlib/Algebra/Polynomial/Inductions.lean,Mathlib/Algebra/Polynomial/Mirror.lean,Mathlib/Algebra/Polynomial/Reverse.lean,Mathlib/Tactic.lean,Mathlib/Tactic/ToNatDegree.lean,scripts/noshake.json |
11 |
2 |
['adomani', 'grunweg'] |
nobody |
390-50588 1 year ago |
390-50588 1 year ago |
0-0 0 seconds |
15823 |
eric-wieser author:eric-wieser |
Quotients of rings in model theory |
---
[](https://gitpod.io/from-referrer/)
|
t-logic
merge-conflict
|
55/13 |
Mathlib/ModelTheory/Algebra/Ring/FreeCommRing.lean,Mathlib/ModelTheory/Syntax.lean |
2 |
1 |
['github-actions'] |
nobody |
390-29151 1 year ago |
390-29151 1 year ago |
0-0 0 seconds |
12178 |
joneugster author:joneugster |
feat(Data/Matrix/Basic): add notation for `m×n`-Matrices |
Introduce the notation `Mat[m,n][R]` for `Matrix (Fin m) (Fin n) R`.
[Zulip thread](https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/Why.20does.20.60Matrix.2Erow.60.20use.20.20.60Unit.60.20instead.20of.20.60Fin.201.60.3F/near/427949223)
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
label:t-algebra$ |
139/135 |
Mathlib/Algebra/Lie/CartanMatrix.lean,Mathlib/Analysis/Complex/UpperHalfPlane/Basic.lean,Mathlib/Data/Matrix/Basic.lean,Mathlib/Data/Matrix/Notation.lean,Mathlib/Data/Matrix/Rank.lean,Mathlib/Data/Matrix/Reflection.lean,Mathlib/GroupTheory/Coxeter/Matrix.lean,Mathlib/LinearAlgebra/Matrix/Adjugate.lean,Mathlib/LinearAlgebra/Matrix/Charpoly/Coeff.lean,Mathlib/LinearAlgebra/Matrix/Determinant.lean,Mathlib/LinearAlgebra/Matrix/SpecialLinearGroup.lean,Mathlib/LinearAlgebra/Matrix/Trace.lean,Mathlib/LinearAlgebra/Matrix/Transvection.lean,Mathlib/LinearAlgebra/PID.lean,Mathlib/LinearAlgebra/Vandermonde.lean,Mathlib/NumberTheory/Modular.lean,Mathlib/NumberTheory/ModularForms/CongruenceSubgroups.lean,Mathlib/NumberTheory/ModularForms/SlashActions.lean,Mathlib/NumberTheory/ModularForms/SlashInvariantForms.lean,Mathlib/NumberTheory/RamificationInertia.lean,Mathlib/RingTheory/SimpleModule.lean,test/matrix.lean |
22 |
9 |
['YaelDillies', 'eric-wieser', 'grunweg', 'joneugster'] |
nobody |
390-6275 1 year ago |
390-10189 1 year ago |
0-0 0 seconds |
12751 |
Command-Master author:Command-Master |
feat: add lemmas for Nat/Bits, Nat/Bitwise and Nat/Size |
Remove `@[simp]` from `Nat.bit_false` and `Nat.bit_true`, as `bit0` and `bit1` are deprecated, and add some lemmas to `Bits`, `Bitwise` and `Size`.
---
[](https://gitpod.io/from-referrer/)
|
t-data
new-contributor
merge-conflict
|
66/7 |
Mathlib/Data/Nat/Bits.lean,Mathlib/Data/Nat/Bitwise.lean,Mathlib/Data/Nat/Multiplicity.lean,Mathlib/Data/Nat/Size.lean |
4 |
26 |
['Command-Master', 'Rida-Hamadani', 'Ruben-VandeVelde', 'YaelDillies', 'github-actions', 'jcommelin'] |
nobody |
389-72639 1 year ago |
395-2481 1 year ago |
54-52408 54 days |
15448 |
urkud author:urkud |
chore(*): deprecate `Option.elim'` |
Use `Option.elim` instead.
---
[](https://gitpod.io/from-referrer/) |
tech debt
merge-conflict
awaiting-author
|
54/50 |
Mathlib/Algebra/BigOperators/Option.lean,Mathlib/Algebra/MvPolynomial/Equiv.lean,Mathlib/Algebra/MvPolynomial/Variables.lean,Mathlib/Analysis/BoxIntegral/Partition/Additive.lean,Mathlib/Analysis/BoxIntegral/Partition/Basic.lean,Mathlib/Analysis/BoxIntegral/Partition/Split.lean,Mathlib/Analysis/Calculus/LagrangeMultipliers.lean,Mathlib/CategoryTheory/Category/PartialFun.lean,Mathlib/Computability/TMToPartrec.lean,Mathlib/Data/Option/Defs.lean,Mathlib/LinearAlgebra/Basis.lean,Mathlib/Logic/Embedding/Set.lean,Mathlib/Logic/Equiv/Basic.lean,Mathlib/MeasureTheory/OuterMeasure/Induced.lean,Mathlib/NumberTheory/Dioph.lean,Mathlib/Topology/Compactness/Paracompact.lean,Mathlib/Topology/LocallyFinite.lean |
17 |
12 |
['Ruben-VandeVelde', 'YaelDillies', 'github-actions', 'grunweg', 'urkud'] |
nobody |
389-61692 1 year ago |
390-50839 1 year ago |
7-18420 7 days |
10349 |
Shamrock-Frost author:Shamrock-Frost |
refactor(CategoryTheory/MorphismProperty) |
We make explicit some of the galois connections/closure operators in the existing MorphismProperty file, rewrite some proofs to take advantage of these structures, and change map/inverseImage by (1) swapping their argument order, for consistency with Set.range and Set.preimage and (2) making "map" perform the strict, evil map while "essMap" (previously called map) forms the closure of the image under isomorphisms. Finally we add `IsMultiplicative` instances for isos/epis/monos, with an eye towards constructing the wide subcategory on these classes of maps.
---
- [x] depends on: #10347
- [ ] depends on: #10348
[](https://gitpod.io/from-referrer/)
|
t-category-theory
merge-conflict
|
474/318 |
Mathlib/CategoryTheory/Localization/Composition.lean,Mathlib/CategoryTheory/Localization/LocalizerMorphism.lean,Mathlib/CategoryTheory/MorphismProperty.lean,Mathlib/Data/Set/Lattice.lean,Mathlib/Order/Closure.lean,Mathlib/Order/Hom/Basic.lean,Mathlib/Order/Hom/CompleteLattice.lean,Mathlib/Order/RelIso/Basic.lean |
8 |
1 |
['leanprover-community-mathlib4-bot'] |
nobody |
387-74922 1 year ago |
430-76042 1 year ago |
0-418 6 minutes |
10350 |
Shamrock-Frost author:Shamrock-Frost |
feat(Data/Setoid): add the operations of taking the equivalence class of an element and of saturating a set wrt an equivalence relation |
I'm open to suggestions about changing the name "saturate", someone on zulip rightly pointed out this is a very overloaded term in math. That said, I think it's unlikely to cause confusion and that there's only one reasonable interpretation in the context of setoids.
---
- [x] depends on: #10347
- [x] depends on: #10348
[](https://gitpod.io/from-referrer/)
|
t-data
merge-conflict
|
169/3 |
Mathlib/Data/Setoid/Basic.lean,Mathlib/Data/Setoid/Partition.lean,Mathlib/Order/Closure.lean |
3 |
1 |
['leanprover-community-mathlib4-bot'] |
nobody |
387-74913 1 year ago |
395-2483 1 year ago |
19-74514 19 days |
13573 |
Shamrock-Frost author:Shamrock-Frost |
feat: add multivariate polynomial modules |
Add a type synonym for multivariate polynomials with coefficients in a module.
---
Multivariate polynomials with module coefficients are sort of silly, but they sometimes show up in commutative algebra (eg in the definition of a quasi regular sequence). Writing this code involved a lot of copy and pasting from `PolynomialModule` and `MvPolynomial`. The API is definitely lacking at this stage but it's a start.
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
awaiting-author
label:t-algebra$ |
691/6 |
Mathlib.lean,Mathlib/Algebra/MvPolynomial/Module/Basic.lean,Mathlib/Algebra/MvPolynomial/Module/MvAEval.lean,Mathlib/Algebra/Polynomial/Module/Basic.lean |
4 |
9 |
['Shamrock-Frost', 'erdOne', 'github-actions'] |
nobody |
387-74893 1 year ago |
393-85488 1 year ago |
39-72739 39 days |
6517 |
MohanadAhmed author:MohanadAhmed |
feat: discrete Fourier transform of a finite sequence |
# Discrete Fourier Transform (DFT) Matrix and DFT of a (finite) sequence
This file defines the `dft` opertaion on a sequence (also a vecotr) and the DFT operation matrix
## Main definitions
- `dft v`: given a sequence (v : (Fin n) → ℂ) we can transform it into a sequence (V : (Fin n) →ℂ)
such that
$$V [p] = ∑_{k = 0}^{N - 1} e^{-j*2πkp/n} v [k]$$
- `idft V` : given a sequence (V : (Fin n) → ℂ) we can transform it into a sequence
(v : (Fin n) → ℂ)
such that
$$v [k] = \frac{1}{N}∑_{p = 0}^{n - 1} e^{j*2πkp/N} v [p]$$
- `dftMatrix n` : the dft matrix of dimensions $n \times n$ with the `k, p` entry equal to
$$Wₙ[k, p] = e^{-j2πkp/n}$$
- `(dftMatrix n)⁻¹` : the idft matrix of dimensions $n \times n$ with the `k, p` entry equal to
$$Wₙ[k, p] = (1/N) e^{j2πkp/n}$$
## Main results
- `dft v = (dftMatrix n) v` : the dft operation on a sequence is the same as the dft matrix applied to the vector
- `idft V = (dftMatrix n)⁻¹ V` : the idft operation on a sequence is the same as the idft matrix applied to the vector
- `dft (idft v) = dft ( idft v) = v` the dft and idft operations are inverses
- `Wₙ = vandermonde (w)` : the dft matrix is vandermonde with `w` being the first row of the dft matrix
- `circulant t = (dftMatrix n)⁻¹ ⬝ diagonal (dft t) ⬝ (dftMatrix n)` : a circulant matrix is diagonalizable by the dft and idft matrix pair.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
awaiting-author
label:t-algebra$ |
294/0 |
Mathlib.lean,Mathlib/LinearAlgebra/Matrix/DFT.lean |
2 |
26 |
['MohanadAhmed', 'ericrbg'] |
nobody |
387-74731 1 year ago |
466-64321 1 year ago |
65-20427 65 days |
13155 |
alreadydone author:alreadydone |
feat(NumberTheory/EllipticDivisibilitySequence): show elliptic relations follow from even-odd recursion |
This PR is centered around the (generalized) elliptic relations (`rel₄`)
$E(a,b,c,d): W_{a+b}W_{a-b}W_{c+d}W_{c-d}=W_{a+c}W_{a-c}W_{b+d}W_{b-d}-W_{a+d}W_{a-d}W_{b+c}W_{b-c}$.
For an integer-indexed sequence W valued in a commutative ring, the relation makes sense only when a,b,c,d are all integers or all half integers. For convenience of formalization, we instead consider integers a,b,c,d of the same parity and divide all subscripts by 2. We extract the subexpression $W_{(a+b)/2}W_{(a-b)/2}$ (which appear six times) as `addMulSub W a b`.
The collection of all $E(a,b,c,d)$ is equivalent to Stange's axiom for elliptic nets (`net`), and the literature (e.g. Silverman) commonly consider only the three-index special case $E(m,n,r,0)$ (`Rel₃`). Important special cases of these relations are
(i) $E(m+1,m,1,0): W_{2m+1}W_1^3=W_{m+2}W_m^3-W_{m+1}^3 W_{m-1}$ (`oddRec`) and
(ii) $E(m+1,m-1,1,0): W_{2m}W_2 W_1^2=W_m(W_{m+2}W_{m-1}^2-W_{m-2}W_{m+1}^2)$ (`evenRec`),
which suffice to uniquely specify $W$ on all positive integers recursively from four initial values $W_1, W_2, W_3, W_4$ (`IsEllSequence.ext`, if $W_1 W_2$ is not a zero divisor). In the usual setting where $W_1=1$ and $W_2\mid W_4$, there does exist a sequence (`normEDS`) satisfying (i) and (ii) given initial values $W_2, W_3$ and $W_4/W_2$. It turns out the same non-zerodivisor condition also guarantees that W is an odd function with $W_0=0$, which naturally extends W to all integers.
The main result of this PR (`rel₄_of_oddRec_evenRec`, `IsEllSequence.of_oddRec_evenRec`) is a purely algebraic proof that the sequence W defined by the single-parameter elliptic relations (i) and (ii) implies all $E(a,b,c,d)$, based on my original argument first published on [Math.SE](https://math.stackexchange.com/a/4903422/12932). It's based on the observation that a nonzerodivisor-multiple of $E(a,b,c,d)$ can be expressed as a linear combination of various $E(a,b,c_\min,d_\min)$ with the two smallest indices fixed at their minimal possible values, which can be transformed (`transf`) to an elliptic relation with smaller `a` (which can be assumed to hold by induction), unless they are of the form (i) or (ii) which hold by assumption. For this argument it's necessary to assume `a > b > c > d ≥ 0` (see `StrictAnti₄` and `Rel₄OfValid`), but it's easy to extend to arbitrary a,b,c,d by symmetry properties of `rel₄` under negation and permutations of indices.
In the subsequent PR #13057, we show all normalized EDSs (`normEDS`), defined using the even-odd recursion (i)-(ii), are elliptic (i.e. satisfy the elliptic relations) divisibility sequences. This PR doesn't directly apply because a normEDS doesn't always satisfy the nonzerodivisor condition, but they are specializations of the universal normEDS, which does satisfy the condition. The technique of reducing to the universal case will be applied many times, and relies on the naturality (`map`) lemmas.
We also change the `ℕ` in the definition `IsDivSequence` to `ℤ` which is more natural given that W is a `ℤ`-indexed sequence.
---
- [x] depends on: #13153
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-number-theory
merge-conflict
awaiting-author
label:t-algebra$ |
565/12 |
Mathlib/NumberTheory/EllipticDivisibilitySequence.lean |
1 |
55 |
['Multramate', 'alreadydone', 'github-actions', 'grunweg', 'leanprover-community-mathlib4-bot'] |
nobody |
382-1935 1 year ago |
382-1935 1 year ago |
26-39367 26 days |
15600 |
adomani author:adomani |
feat: lint also `let` vs `have` |
---
[](https://gitpod.io/from-referrer/)
|
t-linter
merge-conflict
WIP
|
77/26 |
Mathlib/Tactic/Linter/HaveLetLinter.lean,test/HaveLetLinter.lean |
2 |
1 |
['github-actions'] |
nobody |
380-56611 1 year ago |
380-56611 1 year ago |
0-8 8 seconds |
13970 |
adomani author:adomani |
feat: a linter to flag unnecessary uses of `nolint simpNF` |
---
[](https://gitpod.io/from-referrer/)
|
t-linter
merge-conflict
awaiting-author
|
230/0 |
Mathlib.lean,Mathlib/Analysis/CStarAlgebra/Basic.lean,Mathlib/Analysis/Quaternion.lean,Mathlib/CategoryTheory/Comma/Arrow.lean,Mathlib/CategoryTheory/Monoidal/End.lean,Mathlib/Data/NNRat/Defs.lean,Mathlib/Data/Rat/Defs.lean,Mathlib/LinearAlgebra/CliffordAlgebra/Even.lean,Mathlib/LinearAlgebra/CliffordAlgebra/EvenEquiv.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter.lean,Mathlib/Tactic/Linter/UnnecessarySyntax.lean,test/UnnecessarySyntax.lean |
13 |
4 |
['adomani', 'github-actions', 'grunweg', 'leanprover-bot'] |
nobody |
378-79825 1 year ago |
378-79826 1 year ago |
0-0 0 seconds |
15162 |
adomani author:adomani |
feat: checkAsSorry linter |
A very preliminary version of the `checkAsSorry` linter.
It flags declarations whose type is not equal to the 'asSorry'ed one.
[Zulip discussion](https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/Running.20Mathlib.20under.20.60set_option.20debug.2EbyAsSorry.60)
---
[](https://gitpod.io/from-referrer/)
|
t-linter
merge-conflict
|
119/0 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter/CheckAsSorry.lean,test/CheckAsSorry.lean |
4 |
1 |
['github-actions'] |
nobody |
378-78813 1 year ago |
378-78813 1 year ago |
0-0 0 seconds |
14046 |
adomani author:adomani |
test: diff of declarations in lean |
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict
WIP
|
231/2 |
.github/workflows/bors.yml,.github/workflows/build.yml,.github/workflows/build.yml.in,.github/workflows/build_fork.yml,.github/workflows/mk_build_yml.sh,Mathlib/Tactic/Eval.lean,scripts/decls_diff_hybrid.sh,scripts/list_decls.lean |
8 |
2 |
['github-actions'] |
nobody |
374-72327 1 year ago |
374-72327 1 year ago |
0-0 0 seconds |
14038 |
adomani author:adomani |
test/decl diff in lean dev |
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict
WIP
|
231/2 |
.github/workflows/bors.yml,.github/workflows/build.yml,.github/workflows/build.yml.in,.github/workflows/build_fork.yml,.github/workflows/mk_build_yml.sh,Mathlib/Tactic/Eval.lean,scripts/decls_diff_hybrid.sh,scripts/list_decls.lean |
8 |
3 |
['github-actions'] |
nobody |
374-72327 1 year ago |
374-72327 1 year ago |
0-0 0 seconds |
12107 |
yuma-mizuno author:yuma-mizuno |
feat(Mathlib/Tactic/Widget/StringDiagram): support 2-morphisms in bicategories |
---
- [x] depends on: #11080
[](https://gitpod.io/from-referrer/)
|
t-category-theory
t-meta
merge-conflict
|
1158/0 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/CategoryTheory/Coherence.lean,Mathlib/Tactic/Widget/StringDiagram.lean,scripts/noshake.json,test/StringDiagram.lean,widget/src/penrose/monoidal.dsl,widget/src/penrose/monoidal.sty |
8 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
369-67071 1 year ago |
369-67074 1 year ago |
0-0 0 seconds |
15925 |
yuma-mizuno author:yuma-mizuno |
feat(CategoryTheory/Monoida): proof producing coherence tactic |
---
[](https://gitpod.io/from-referrer/)
|
t-category-theory
t-meta
merge-conflict
|
5018/265 |
Mathlib.lean,Mathlib/CategoryTheory/Bicategory/Adjunction.lean,Mathlib/CategoryTheory/Bicategory/Kan/Adjunction.lean,Mathlib/CategoryTheory/Monoidal/Braided/Basic.lean,Mathlib/CategoryTheory/Monoidal/CoherenceLemmas.lean,Mathlib/CategoryTheory/Monoidal/Opposite.lean,Mathlib/CategoryTheory/Monoidal/Rigid/Basic.lean,Mathlib/CategoryTheory/Monoidal/Rigid/Braided.lean,Mathlib/Tactic.lean,Mathlib/Tactic/CategoryTheory/BicategoricalComp.lean,Mathlib/Tactic/CategoryTheory/Bicategory/Normalize.lean,Mathlib/Tactic/CategoryTheory/Bicategory/PureCoherence.lean,Mathlib/Tactic/CategoryTheory/Coherence.lean,Mathlib/Tactic/CategoryTheory/Coherence/Basic.lean,Mathlib/Tactic/CategoryTheory/Coherence/Datatypes.lean,Mathlib/Tactic/CategoryTheory/Coherence/Normalize.lean,Mathlib/Tactic/CategoryTheory/Coherence/PureCoherence.lean,Mathlib/Tactic/CategoryTheory/CoherenceNew.lean,Mathlib/Tactic/CategoryTheory/Monoidal.lean,Mathlib/Tactic/CategoryTheory/Monoidal/Basic.lean,Mathlib/Tactic/CategoryTheory/Monoidal/Datatypes.lean,Mathlib/Tactic/CategoryTheory/Monoidal/Normalize.lean,Mathlib/Tactic/CategoryTheory/Monoidal/PureCoherence.lean,Mathlib/Tactic/CategoryTheory/MonoidalComp.lean,Mathlib/Tactic/Widget/StringDiagram.lean,lake-manifest.json,scripts/noshake.json,test/CategoryTheory/Bicategory.lean,test/CategoryTheory/Coherence.lean,test/CategoryTheory/CoherenceNew.lean,test/CategoryTheory/Monoidal.lean,test/CategoryTheory/Monoidal/Basic.lean,test/CategoryTheory/Monoidal/Normalize.lean,test/CategoryTheory/MonoidalComp.lean,test/StringDiagram.lean |
35 |
n/a |
['github-actions'] |
nobody |
369-27208 1 year ago |
unknown |
unknown |
6475 |
joneugster author:joneugster |
refactor(LinearAlgebra/Span): replace ∙ with • as notation for `span R {x}` |
Change the notation for `Submodule.span R {x}` from `R ∙ x` to the bullet `R • x`, which is also used for scalar multiplication.
---
(this was an experiment originating from a [Zulip discussion](https://leanprover.zulipchat.com/#narrow/stream/270676-lean4/topic/.2E.C2.B7.E2.AC.9D.20.5Brant.5D), I don't have a clear opinion if this is actually a desired thing to do...)
Generally this works and Lean seems to do fine figuring out the difference between `r • x` and `R • x` (The former is scalar multiplication in an `R`-module `M`, the latter is the `Submodule R M` generated by `x`).
Encountered a few regressions that should be considered (the first two might be also bugs that could be looked at independently):
1. `(· • ·)`, and general simple function syntax, does not work as notation for `HSMul.hSMul` anymore. For this reason, I introduced the notation `scoped` to minimise the effect of this. Now it's only a problem if you `open Span`. Note that `fun x₁ x₂ ↦ x₁ • x₂` works flawlessly all the time.
4. `change` and `convert` have troubles to deal with the two competing notations. `have := _; convert this` works.
5. `R • x - y` is not valid anymore and needs parentheses: `R • (x - y)`. I do think this actually helps readability, so I don't mind.
[](https://gitpod.io/from-referrer/)
|
t-algebra
RFC
merge-conflict
label:t-algebra$ |
323/240 |
Mathlib/Algebra/Algebra/Operations.lean,Mathlib/Algebra/Algebra/Subalgebra/Basic.lean,Mathlib/Algebra/Lie/Engel.lean,Mathlib/Algebra/Lie/Normalizer.lean,Mathlib/Algebra/Module/PID.lean,Mathlib/Algebra/Module/Torsion.lean,Mathlib/Analysis/InnerProductSpace/Basic.lean,Mathlib/Analysis/InnerProductSpace/GramSchmidtOrtho.lean,Mathlib/Analysis/InnerProductSpace/Orthogonal.lean,Mathlib/Analysis/InnerProductSpace/PiL2.lean,Mathlib/Analysis/InnerProductSpace/Projection.lean,Mathlib/Analysis/InnerProductSpace/TwoDim.lean,Mathlib/Analysis/NormedSpace/ContinuousLinearMap.lean,Mathlib/Analysis/NormedSpace/HahnBanach/Extension.lean,Mathlib/Analysis/NormedSpace/OperatorNorm.lean,Mathlib/Data/ZMod/Quotient.lean,Mathlib/Geometry/Euclidean/Angle/Oriented/Basic.lean,Mathlib/Geometry/Euclidean/Inversion/Calculus.lean,Mathlib/Geometry/Euclidean/MongePoint.lean,Mathlib/Geometry/Euclidean/PerpBisector.lean,Mathlib/Geometry/Euclidean/Sphere/SecondInter.lean,Mathlib/Geometry/Manifold/Instances/Sphere.lean,Mathlib/LinearAlgebra/AffineSpace/AffineSubspace.lean,Mathlib/LinearAlgebra/AffineSpace/FiniteDimensional.lean,Mathlib/LinearAlgebra/BilinearForm.lean,Mathlib/LinearAlgebra/DFinsupp.lean,Mathlib/LinearAlgebra/Dimension.lean,Mathlib/LinearAlgebra/FiniteDimensional.lean,Mathlib/LinearAlgebra/LinearIndependent.lean,Mathlib/LinearAlgebra/LinearPMap.lean,Mathlib/LinearAlgebra/ProjectiveSpace/Basic.lean,Mathlib/LinearAlgebra/QuadraticForm/Basic.lean,Mathlib/LinearAlgebra/Quotient.lean,Mathlib/LinearAlgebra/SesquilinearForm.lean,Mathlib/LinearAlgebra/Span.lean,Mathlib/MeasureTheory/Integral/Periodic.lean,Mathlib/RingTheory/Coprime/Ideal.lean,Mathlib/RingTheory/Finiteness.lean,Mathlib/RingTheory/Ideal/AssociatedPrime.lean,Mathlib/RingTheory/Ideal/IdempotentFG.lean,Mathlib/RingTheory/Noetherian.lean,Mathlib/Topology/Instances/AddCircle.lean |
42 |
3 |
['eric-wieser', 'joneugster', 'leanprover-bot'] |
nobody |
368-5564 1 year ago |
368-5564 1 year ago |
0-0 0 seconds |
7545 |
shuxuezhuyi author:shuxuezhuyi |
feat: APIs of `Function.extend f g e'` when `f` is injective |
We characterizes `range g`, `Injective g`, `Surjective g` and `Bijective g` in terms of `extend f g e'`.
---
[](https://gitpod.io/from-referrer/)
|
t-logic
merge-conflict
awaiting-author
|
50/0 |
Mathlib.lean,Mathlib/Logic/Function/ApiForExtend.lean |
2 |
1 |
['fpvandoorn'] |
nobody |
367-21100 1 year ago |
367-21100 1 year ago |
32-30254 32 days |
12632 |
urkud author:urkud |
feat(List/OffDiag): new file |
---
[](https://gitpod.io/from-referrer/)
|
t-data
merge-conflict
awaiting-author
|
184/3 |
Mathlib.lean,Mathlib/Data/List/Basic.lean,Mathlib/Data/List/Enum.lean,Mathlib/Data/List/EraseIdx.lean,Mathlib/Data/List/OffDiag.lean |
5 |
3 |
['eric-wieser', 'github-actions', 'urkud'] |
nobody |
363-78315 11 months ago |
363-78315 11 months ago |
0-0 0 seconds |
16658 |
adomani author:adomani |
add tips file |
---
[](https://gitpod.io/from-referrer/)
|
test-ci
merge-conflict
awaiting-author
WIP
|
51/508 |
.github/build.in.yml,.github/workflows/bors.yml,.github/workflows/build.yml,.github/workflows/build_fork.yml,scripts/Tips.lean |
5 |
1 |
['github-actions'] |
nobody |
363-50033 11 months ago |
363-50033 11 months ago |
0-0 0 seconds |
14078 |
Ruben-VandeVelde author:Ruben-VandeVelde |
feat(CI): continue after mk_all fails |
---
[](https://gitpod.io/from-referrer/)
|
CI
merge-conflict
awaiting-author
|
43/0 |
.github/workflows/bors.yml,.github/workflows/build.yml,.github/workflows/build.yml.in,.github/workflows/build_fork.yml,Mathlib/Data/Nat/Test.lean |
5 |
2 |
['bryangingechen', 'github-actions'] |
nobody |
363-30333 11 months ago |
363-30333 11 months ago |
0-0 0 seconds |
11800 |
JADekker author:JADekker |
feat : Define KappaLindelöf spaces |
Define KappaLindelöf spaces by following the first one-third of the API for Lindelöf spaces. The remainder will be added in a future PR.
---
[](https://gitpod.io/from-referrer/)
|
awaiting-zulip
t-topology
merge-conflict
please-adopt
|
301/2 |
Mathlib.lean,Mathlib/Topology/Compactness/KappaLindelof.lean,Mathlib/Topology/Compactness/Lindelof.lean |
3 |
38 |
['ADedecker', 'JADekker', 'PatrickMassot', 'StevenClontz', 'adomani', 'github-actions', 'grunweg', 'kim-em', 'urkud'] |
nobody |
362-21110 11 months ago |
362-43085 11 months ago |
119-10687 119 days |
11283 |
hmonroe author:hmonroe |
feat(ModelTheory/Satisfiability): define theory with independent sentence |
---
[](https://gitpod.io/from-referrer/)
|
t-logic
merge-conflict
WIP
|
8/0 |
Mathlib/ModelTheory/Satisfiability.lean |
1 |
2 |
['fpvandoorn', 'hmonroe'] |
nobody |
361-887 11 months ago |
361-887 11 months ago |
3-5240 3 days |
16914 |
siddhartha-gadgil author:siddhartha-gadgil |
Loogle syntax with non-reserved |
This is PR mainly to test that loogle syntax does not break stuff downstream
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict
WIP
|
4/4 |
lake-manifest.json,lakefile.lean |
2 |
1 |
['github-actions'] |
nobody |
358-75896 11 months ago |
358-75896 11 months ago |
0-14835 4 hours |
10075 |
dupuisf author:dupuisf |
refactor: generalize `MonoidHom.ker` and `MonoidHom.range` to `MonoidHomClass` |
With this refactor, `MonoidHom.ker` and `MonoidHom.range` will be defined for any `MonoidHomClass` type, not just `MonoidHom`s. This brings the design in line with `LinearMap.ker`/`range` and `MonoidHom.mker`/`mrange`. `Subgroup.map`/`comap` are also generalized.
As with those previous refactors, the main drawback is the loss of dot notation in many cases. Other than that, the impact is fairly minor given that this is happening is rather basic files.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
awaiting-author
label:t-algebra$ |
464/389 |
Mathlib/Algebra/Category/GroupCat/Abelian.lean,Mathlib/Algebra/Category/GroupCat/Basic.lean,Mathlib/Algebra/Category/GroupCat/Colimits.lean,Mathlib/Algebra/Category/GroupCat/EpiMono.lean,Mathlib/Algebra/Category/GroupCat/Images.lean,Mathlib/Algebra/Category/GroupCat/Kernels.lean,Mathlib/Algebra/Category/GroupCat/Limits.lean,Mathlib/Algebra/Homology/ShortComplex/Ab.lean,Mathlib/Analysis/Normed/Group/Basic.lean,Mathlib/Analysis/Normed/Group/Hom.lean,Mathlib/Data/ZMod/Basic.lean,Mathlib/Data/ZMod/Quotient.lean,Mathlib/FieldTheory/PolynomialGaloisGroup.lean,Mathlib/GroupTheory/Abelianization.lean,Mathlib/GroupTheory/CoprodI.lean,Mathlib/GroupTheory/Coset.lean,Mathlib/GroupTheory/Finiteness.lean,Mathlib/GroupTheory/FreeGroup/Basic.lean,Mathlib/GroupTheory/GroupAction/Quotient.lean,Mathlib/GroupTheory/HNNExtension.lean,Mathlib/GroupTheory/Index.lean,Mathlib/GroupTheory/Nilpotent.lean,Mathlib/GroupTheory/NoncommPiCoprod.lean,Mathlib/GroupTheory/PGroup.lean,Mathlib/GroupTheory/Perm/Sign.lean,Mathlib/GroupTheory/Perm/Subgroup.lean,Mathlib/GroupTheory/PushoutI.lean,Mathlib/GroupTheory/QuotientGroup.lean,Mathlib/GroupTheory/SchurZassenhaus.lean,Mathlib/GroupTheory/SemidirectProduct.lean,Mathlib/GroupTheory/Solvable.lean,Mathlib/GroupTheory/SpecificGroups/Alternating.lean,Mathlib/GroupTheory/SpecificGroups/Cyclic.lean,Mathlib/GroupTheory/Subgroup/Basic.lean,Mathlib/GroupTheory/Subgroup/Finite.lean,Mathlib/GroupTheory/Subgroup/Saturated.lean,Mathlib/GroupTheory/Subgroup/ZPowers.lean,Mathlib/GroupTheory/Sylow.lean,Mathlib/GroupTheory/Torsion.lean,Mathlib/GroupTheory/Transfer.lean,Mathlib/LinearAlgebra/Alternating/DomCoprod.lean,Mathlib/LinearAlgebra/Basic.lean,Mathlib/LinearAlgebra/Matrix/Determinant.lean,Mathlib/MeasureTheory/Function/LpSpace.lean,Mathlib/NumberTheory/ModularForms/CongruenceSubgroups.lean,Mathlib/RingTheory/ClassGroup.lean,Mathlib/RingTheory/DedekindDomain/SelmerGroup.lean,Mathlib/RingTheory/Valuation/ValuationSubring.lean,Mathlib/Topology/Algebra/OpenSubgroup.lean,Mathlib/Topology/Algebra/UniformGroup.lean,Mathlib/Topology/Instances/AddCircle.lean |
51 |
2 |
['dupuisf', 'urkud'] |
nobody |
358-73785 11 months ago |
359-18650 11 months ago |
8-14499 8 days |
10991 |
thorimur author:thorimur |
feat: `tfae` block tactic |
This PR introduces `tfae` block tactic syntax:
```lean
tfae
1 → 2 := /- proof of `P₁ → P₂` -/
2 → 3 := /- proof of `P₂ → P₃` -/
3 → 1 := /- proof of `P₃ → P₁` -/
```
Like the recent change to `tfae_have`, this syntax also supports all sorts of matching that `have` itself supports:
```lean
tfae
2 → 3
| h₂ => /- proof of `P₃` -/
3 → 1 -- given `P₁ := ∀(a : A), (b : B), (c : C), X`:
| h₃, a, b, c => /- proof of `X` -/
⟨h_mp, h_mpr⟩ : 1 ↔ 2 := /- proof of `P₁ ↔ P₂`; puts `h_mp : P₁ → P₂`, `h_mpr : P₂ → P₁` in the lctx -/
```
This initial implementation is currently very simple, and relies on `tfae_have` and `tfae_finish`. Although we intend to migrate away from that syntax, this PR does not remove support for it or deprecate `tfae_have`/`tfae_finish` in any way; migration (but not deprecation) is done in #11003.
---
- [ ] depends on: #10653
- [x] depends on: #10994
[](https://gitpod.io/from-referrer/)
|
t-meta
merge-conflict
modifies-tactic-syntax
WIP
|
392/124 |
Mathlib/Tactic/TFAE.lean,scripts/noshake.json,test/tfae.lean |
3 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
358-13150 11 months ago |
358-13150 11 months ago |
0-0 0 seconds |
16464 |
Parcly-Taxel author:Parcly-Taxel |
chore: deprecate `Nat.(case_)strong_induction_on` |
…in favour of the now-renamed `Nat.(case)strongInductionOn` in core. |
tech debt
merge-conflict
|
54/56 |
Archive/Imo/Imo1981Q3.lean,Mathlib/Algebra/ContinuedFractions/Computation/Approximations.lean,Mathlib/Algebra/ContinuedFractions/Computation/TerminatesIffRat.lean,Mathlib/Algebra/ContinuedFractions/ConvergentsEquiv.lean,Mathlib/Algebra/Polynomial/Derivative.lean,Mathlib/Algebra/Polynomial/Lifts.lean,Mathlib/Analysis/Analytic/Basic.lean,Mathlib/Analysis/Calculus/ContDiff/Bounds.lean,Mathlib/Analysis/Hofer.lean,Mathlib/Analysis/SpecificLimits/Normed.lean,Mathlib/Combinatorics/Derangements/Finite.lean,Mathlib/Combinatorics/Enumerative/Catalan.lean,Mathlib/Combinatorics/Hall/Finite.lean,Mathlib/Combinatorics/SetFamily/AhlswedeZhang.lean,Mathlib/Computability/Primrec.lean,Mathlib/Data/Fintype/Basic.lean,Mathlib/Data/Fintype/Card.lean,Mathlib/Data/Nat/Choose/Central.lean,Mathlib/Data/Nat/Defs.lean,Mathlib/Data/Nat/Digits.lean,Mathlib/Data/Nat/Log.lean,Mathlib/FieldTheory/Separable.lean,Mathlib/LinearAlgebra/Eigenspace/Triangularizable.lean,Mathlib/LinearAlgebra/Multilinear/Basic.lean,Mathlib/NumberTheory/BernoulliPolynomials.lean,Mathlib/NumberTheory/DiophantineApproximation.lean,Mathlib/NumberTheory/Pell.lean,Mathlib/NumberTheory/Primorial.lean,Mathlib/Order/Fin/Basic.lean,Mathlib/RingTheory/Adjoin/PowerBasis.lean,Mathlib/RingTheory/LittleWedderburn.lean,Mathlib/RingTheory/Polynomial/Basic.lean,Mathlib/RingTheory/Polynomial/Cyclotomic/Basic.lean,Mathlib/RingTheory/Polynomial/Cyclotomic/Eval.lean,Mathlib/RingTheory/Polynomial/Eisenstein/IsIntegral.lean,Mathlib/RingTheory/Polynomial/Nilpotent.lean,Mathlib/RingTheory/PowerSeries/Basic.lean,Mathlib/RingTheory/QuotientNilpotent.lean,Mathlib/RingTheory/WittVector/Defs.lean,Mathlib/RingTheory/WittVector/Frobenius.lean,Mathlib/RingTheory/WittVector/StructurePolynomial.lean,Mathlib/SetTheory/Surreal/Dyadic.lean,Mathlib/Topology/Metrizable/Uniformity.lean |
43 |
13 |
['Parcly-Taxel', 'b-mehta', 'github-actions', 'jcommelin'] |
nobody |
357-61195 11 months ago |
357-61195 11 months ago |
8-1989 8 days |
8118 |
iwilare author:iwilare |
feat(CategoryTheory): add dinatural transformations |
A starting point to define [dinatural transformations](https://ncatlab.org/nlab/show/dinatural+transformation).
This is my first PR so style comments and improvements are very welcome!
---
[](https://gitpod.io/from-referrer/)
|
t-category-theory
merge-conflict
awaiting-author
|
147/7 |
Mathlib.lean,Mathlib/CategoryTheory/DinatTrans.lean,Mathlib/CategoryTheory/Functor/Category.lean,Mathlib/CategoryTheory/Products/Bifunctor.lean |
4 |
49 |
['Shamrock-Frost', 'github-actions', 'iwilare', 'joelriou'] |
Shamrock-Frost assignee:Shamrock-Frost |
354-11782 11 months ago |
354-11783 11 months ago |
21-9462 21 days |
17110 |
FR-vdash-bot author:FR-vdash-bot |
chore: deprecate some lemmas about equality |
These lemmas were upstreamed to Batteries in https://github.com/leanprover-community/batteries/pull/465.
---
- [ ] depends on: https://github.com/leanprover-community/batteries/pull/957
[](https://gitpod.io/from-referrer/)
|
blocked-by-batt-PR
merge-conflict
|
20/16 |
Mathlib/Combinatorics/SimpleGraph/Walk.lean,Mathlib/Data/Nat/Bitwise.lean,Mathlib/Logic/Basic.lean,Mathlib/Logic/Equiv/Basic.lean,Mathlib/Tactic/CC/Addition.lean,lake-manifest.json |
6 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
349-60969 11 months ago |
349-60971 11 months ago |
0-0 0 seconds |
17171 |
FR-vdash-bot author:FR-vdash-bot |
test extends carrier and property |
---
We need https://github.com/leanprover/lean4/issues/2666 ...
[](https://gitpod.io/from-referrer/)
|
merge-conflict |
433/309 |
Mathlib/Algebra/Algebra/NonUnitalSubalgebra.lean,Mathlib/Algebra/Algebra/Subalgebra/Basic.lean,Mathlib/Algebra/Algebra/Subalgebra/Directed.lean,Mathlib/Algebra/DirectSum/Decomposition.lean,Mathlib/Algebra/Field/Subfield.lean,Mathlib/Algebra/Group/Subgroup/Basic.lean,Mathlib/Algebra/Group/Subgroup/MulOpposite.lean,Mathlib/Algebra/Group/Submonoid/Basic.lean,Mathlib/Algebra/Group/Submonoid/MulOpposite.lean,Mathlib/Algebra/Group/Submonoid/Pointwise.lean,Mathlib/Algebra/Group/Submonoid/Units.lean,Mathlib/Algebra/Group/Subsemigroup/Basic.lean,Mathlib/Algebra/Group/Subsemigroup/Operations.lean,Mathlib/Algebra/Module/Submodule/Basic.lean,Mathlib/Algebra/Module/Submodule/Lattice.lean,Mathlib/Algebra/Module/Submodule/Map.lean,Mathlib/Algebra/Module/Submodule/Pointwise.lean,Mathlib/Algebra/Ring/Subring/Basic.lean,Mathlib/Algebra/Ring/Subsemiring/Basic.lean,Mathlib/Algebra/Ring/Subsemiring/MulOpposite.lean,Mathlib/Algebra/Ring/Subsemiring/Order.lean,Mathlib/Algebra/Star/Subalgebra.lean,Mathlib/Algebra/Star/Subsemiring.lean,Mathlib/Data/Complex/Module.lean,Mathlib/Data/SetLike/Basic.lean,Mathlib/Deprecated/Subfield.lean,Mathlib/Deprecated/Subgroup.lean,Mathlib/Deprecated/Submonoid.lean,Mathlib/Deprecated/Subring.lean,Mathlib/FieldTheory/IntermediateField/Basic.lean,Mathlib/GroupTheory/ArchimedeanDensely.lean,Mathlib/GroupTheory/DoubleCoset.lean,Mathlib/GroupTheory/Finiteness.lean,Mathlib/GroupTheory/GroupAction/SubMulAction.lean,Mathlib/LinearAlgebra/AffineSpace/AffineSubspace.lean,Mathlib/LinearAlgebra/Span.lean,Mathlib/RingTheory/Ideal/Operations.lean,Mathlib/RingTheory/NonUnitalSubring/Basic.lean,Mathlib/RingTheory/NonUnitalSubsemiring/Basic.lean,Mathlib/SetTheory/Cardinal/Subfield.lean,Mathlib/Topology/Algebra/Algebra.lean,Mathlib/Topology/Algebra/OpenSubgroup.lean |
42 |
1 |
['github-actions'] |
nobody |
349-56875 11 months ago |
349-56875 11 months ago |
0-0 0 seconds |
7516 |
ADedecker author:ADedecker |
perf: use `abbrev` to prevent unifying useless data |
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict
WIP
|
4/3 |
Mathlib/Topology/ContinuousFunction/Bounded.lean |
1 |
3 |
['ADedecker', 'leanprover-bot', 'mattrobball'] |
nobody |
348-28535 11 months ago |
348-28535 11 months ago |
0-0 0 seconds |
17127 |
FR-vdash-bot author:FR-vdash-bot |
chore: remove global `Quotient.mk` `⟦·⟧` notation |
---
Merge this PR when we are ready to migrate to `QuotLike` API (#16421).
[](https://gitpod.io/from-referrer/)
|
t-data
merge-conflict
|
137/2 |
Counterexamples/Pseudoelement.lean,Mathlib/Algebra/Associated/Basic.lean,Mathlib/Algebra/BigOperators/Group/Finset.lean,Mathlib/Algebra/Group/Conj.lean,Mathlib/Algebra/GroupWithZero/NonZeroDivisors.lean,Mathlib/Algebra/Order/CauSeq/Completion.lean,Mathlib/Algebra/Quandle.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Jacobian.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Projective.lean,Mathlib/AlgebraicTopology/FundamentalGroupoid/Basic.lean,Mathlib/AlgebraicTopology/FundamentalGroupoid/FundamentalGroup.lean,Mathlib/AlgebraicTopology/FundamentalGroupoid/InducedMaps.lean,Mathlib/AlgebraicTopology/FundamentalGroupoid/Product.lean,Mathlib/AlgebraicTopology/FundamentalGroupoid/SimplyConnected.lean,Mathlib/CategoryTheory/Abelian/Pseudoelements.lean,Mathlib/CategoryTheory/Limits/Shapes/SingleObj.lean,Mathlib/CategoryTheory/Monoidal/Free/Basic.lean,Mathlib/CategoryTheory/Monoidal/Free/Coherence.lean,Mathlib/CategoryTheory/Skeletal.lean,Mathlib/Data/Finset/Card.lean,Mathlib/Data/Fintype/List.lean,Mathlib/Data/Fintype/Quotient.lean,Mathlib/Data/Multiset/Basic.lean,Mathlib/Data/QPF/Multivariate/Constructions/Fix.lean,Mathlib/Data/QPF/Univariate/Basic.lean,Mathlib/Data/Quot.lean,Mathlib/Data/Real/Basic.lean,Mathlib/Data/Set/Finite.lean,Mathlib/Data/Set/Image.lean,Mathlib/Data/Setoid/Basic.lean,Mathlib/GroupTheory/GroupAction/Basic.lean,Mathlib/GroupTheory/GroupAction/Quotient.lean,Mathlib/LinearAlgebra/Dual.lean,Mathlib/LinearAlgebra/Ray.lean,Mathlib/Logic/Encodable/Basic.lean,Mathlib/Logic/Equiv/Basic.lean,Mathlib/ModelTheory/DirectLimit.lean,Mathlib/ModelTheory/Fraisse.lean,Mathlib/ModelTheory/Quotients.lean,Mathlib/NumberTheory/NumberField/CanonicalEmbedding/FundamentalCone.lean,Mathlib/NumberTheory/NumberField/Embeddings.lean,Mathlib/NumberTheory/NumberField/Units/DirichletTheorem.lean,Mathlib/NumberTheory/Padics/PadicIntegers.lean,Mathlib/NumberTheory/Padics/PadicNumbers.lean,Mathlib/Order/RelIso/Basic.lean,Mathlib/RepresentationTheory/Action/Concrete.lean,Mathlib/SetTheory/Cardinal/Basic.lean,Mathlib/SetTheory/Cardinal/Ordinal.lean,Mathlib/SetTheory/Game/Basic.lean,Mathlib/SetTheory/Game/Birthday.lean,Mathlib/SetTheory/Game/Impartial.lean,Mathlib/SetTheory/Game/Ordinal.lean,Mathlib/SetTheory/Game/State.lean,Mathlib/SetTheory/Lists.lean,Mathlib/SetTheory/Ordinal/Arithmetic.lean,Mathlib/SetTheory/Ordinal/Basic.lean,Mathlib/SetTheory/Surreal/Basic.lean,Mathlib/SetTheory/Surreal/Dyadic.lean,Mathlib/SetTheory/Surreal/Multiplication.lean,Mathlib/SetTheory/ZFC/Basic.lean,Mathlib/SetTheory/ZFC/Rank.lean,Mathlib/Topology/Connected/PathConnected.lean,Mathlib/Topology/Homotopy/HomotopyGroup.lean,Mathlib/Topology/Homotopy/Path.lean,Mathlib/Topology/Homotopy/Product.lean,Mathlib/Topology/MetricSpace/GromovHausdorff.lean,Mathlib/Topology/UniformSpace/Separation.lean,test/interactiveUnfold.lean |
68 |
1 |
['github-actions'] |
nobody |
348-23578 11 months ago |
348-23578 11 months ago |
4-72805 4 days |
14712 |
FR-vdash-bot author:FR-vdash-bot |
perf: change instance priority and order about `OfNat` |
---
[](https://gitpod.io/from-referrer/)
|
slow-typeclass-synthesis
t-algebra
merge-conflict
delegated
label:t-algebra$ |
49/20 |
Mathlib/Algebra/Group/Nat.lean,Mathlib/Algebra/Group/ZeroOne.lean,Mathlib/Algebra/Homology/Embedding/Basic.lean,Mathlib/Algebra/Tropical/Basic.lean,Mathlib/Data/BitVec.lean,Mathlib/Data/Nat/Cast/Defs.lean,Mathlib/Data/Rat/Defs.lean,Mathlib/Data/UInt.lean,Mathlib/NumberTheory/ArithmeticFunction.lean |
9 |
24 |
['FR-vdash-bot', 'MichaelStollBayreuth', 'eric-wieser', 'github-actions', 'j-loreaux', 'leanprover-bot', 'mathlib-bors'] |
nobody |
342-131 11 months ago |
344-23607 11 months ago |
20-15089 20 days |
11500 |
mcdoll author:mcdoll |
refactor(Topology/Algebra/Module/WeakDual): Clean up |
- Move `Dual` and `dualPairing` lower in the import-hierachy
- deduplicate `dualPairing`
- Bundle continuity statements to `CLM`s.
- Make `WeakDual` and `WeakSpace` reducible
- Remove `refine'` in favor of `refine`
---
Cleaning up `Analysis/NormedSpace/WeakDual` will be done in a second PR
[](https://gitpod.io/from-referrer/)
|
t-topology
merge-conflict
awaiting-author
|
227/179 |
Mathlib.lean,Mathlib/Analysis/Fourier/RiemannLebesgueLemma.lean,Mathlib/Analysis/InnerProductSpace/Adjoint.lean,Mathlib/Analysis/InnerProductSpace/Dual.lean,Mathlib/Analysis/LocallyConvex/Polar.lean,Mathlib/Analysis/NormedSpace/Dual.lean,Mathlib/Analysis/NormedSpace/WeakDual.lean,Mathlib/Analysis/VonNeumannAlgebra/Basic.lean,Mathlib/MeasureTheory/Function/AEEqOfIntegral.lean,Mathlib/MeasureTheory/Measure/FiniteMeasure.lean,Mathlib/Topology/Algebra/Module/CharacterSpace.lean,Mathlib/Topology/Algebra/Module/Dual.lean,Mathlib/Topology/Algebra/Module/WeakDual.lean,docs/overview.yaml,docs/undergrad.yaml |
15 |
14 |
['ADedecker', 'grunweg', 'j-loreaux', 'kkytola', 'mathlib-bors', 'mcdoll'] |
nobody |
340-22074 11 months ago |
340-22074 11 months ago |
46-5572 46 days |
5995 |
FR-vdash-bot author:FR-vdash-bot |
feat: add APIs about `Quotient.choice` |
Some docs in this PR refer to the definition in #5576.
---
[](https://gitpod.io/from-referrer/)
|
t-data
RFC
merge-conflict
awaiting-author
|
76/6 |
Mathlib/Data/Quot.lean |
1 |
3 |
['FR-vdash-bot', 'YaelDillies', 'gebner'] |
eric-wieser assignee:eric-wieser |
338-68720 11 months ago |
338-68720 11 months ago |
285-35716 285 days |
8029 |
alreadydone author:alreadydone |
refactor: Homotopy between Functions not ContinuousMaps |
This allows talking about homotopies without needing to supply proofs of continuity for the two ends. This for example simplifies the definition of H-spaces.
Of course, if a homotopy exists between two functions, those two functions are automatically continuous because they are restrictions of the homotopy (which is continuous) to subspaces.
`Homotopy.refl` still needs a continuous map as input, and `Homotopic` is only an equivalence relation when restricted to ContinuousMap.
---
TODO: fix docstrings
[](https://gitpod.io/from-referrer/)
|
t-topology
RFC
merge-conflict
|
246/250 |
Mathlib/AlgebraicTopology/FundamentalGroupoid/InducedMaps.lean,Mathlib/Topology/Homotopy/Basic.lean,Mathlib/Topology/Homotopy/Contractible.lean,Mathlib/Topology/Homotopy/Equiv.lean,Mathlib/Topology/Homotopy/HSpaces.lean,Mathlib/Topology/Homotopy/HomotopyGroup.lean,Mathlib/Topology/Homotopy/Path.lean,Mathlib/Topology/Homotopy/Product.lean |
8 |
3 |
['alreadydone', 'urkud'] |
nobody |
338-52383 11 months ago |
430-76042 1 year ago |
9-20043 9 days |
14619 |
Command-Master author:Command-Master |
chore: Merge `Trunc` to `Squash` |
Remove `Trunc` and use `Squash` instead
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
merge-conflict
WIP
|
197/211 |
Mathlib/CategoryTheory/EpiMono.lean,Mathlib/CategoryTheory/Preadditive/Biproducts.lean,Mathlib/Data/DFinsupp/Basic.lean,Mathlib/Data/Fintype/Basic.lean,Mathlib/Data/Fintype/Card.lean,Mathlib/Data/Fintype/Option.lean,Mathlib/Data/Fintype/Perm.lean,Mathlib/Data/Fintype/Quotient.lean,Mathlib/Data/Quot.lean,Mathlib/Data/Semiquot.lean,Mathlib/GroupTheory/Perm/Cycle/Factors.lean,Mathlib/GroupTheory/Perm/Sign.lean,Mathlib/Logic/Equiv/List.lean |
13 |
3 |
['Command-Master', 'github-actions', 'vihdzp'] |
nobody |
336-14661 11 months ago |
420-72805 1 year ago |
0-0 0 seconds |
13156 |
erdOne author:erdOne |
refactor(Algebra/Module/LocalizedModule): Redefine `LocalizedModule` in terms of `OreLocalization`. |
---
- [x] depends on: #13151
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
label:t-algebra$ |
519/628 |
Mathlib.lean,Mathlib/Algebra/Module/LocalizedModule.lean,Mathlib/AlgebraicGeometry/Modules/Tilde.lean,Mathlib/RingTheory/DedekindDomain/Different.lean,Mathlib/RingTheory/Localization/BaseChange.lean,Mathlib/RingTheory/OreLocalization/Basic.lean,Mathlib/RingTheory/OreLocalization/Module.lean,Mathlib/RingTheory/OreLocalization/Ring.lean |
8 |
4 |
['github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'mattrobball'] |
nobody |
333-75860 10 months ago |
333-75860 10 months ago |
51-84473 51 days |
16348 |
urkud author:urkud |
refactor(Topology): require `LinearOrder` with `OrderTopology` |
While the definition formally makes sense for a preorder,
this topology is usually not the right one for a non-linear order (e.g., `Real × Real`).
See [Zulip thread](https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/Open.20Ioi)
---
This PR doesn't cleanup any API, I'm going to do it in a later PR.
[](https://gitpod.io/from-referrer/)
|
t-order
t-topology
merge-conflict
awaiting-author
|
33/46 |
Mathlib/Analysis/Asymptotics/SuperpolynomialDecay.lean,Mathlib/Topology/Algebra/Order/LiminfLimsup.lean,Mathlib/Topology/Instances/Sign.lean,Mathlib/Topology/Order/Basic.lean,Mathlib/Topology/Order/Filter.lean,Mathlib/Topology/Order/MonotoneContinuity.lean |
6 |
10 |
['YaelDillies', 'github-actions', 'jcommelin', 'urkud'] |
nobody |
333-75484 10 months ago |
333-75484 10 months ago |
3-83049 3 days |
16984 |
hrmacbeth author:hrmacbeth |
feat: extend `module` tactic to handle multiple rings, not strictly ordered by inclusion |
The `module` tactic currently in Mathlib handles scalars from multiple rings, but only if for any two rings `R` and `S` which appear, either `R` is an algebra over `S` or vice versa. This PR extends the tactic by providing a syntax `module T`, which will handle scalars from any ring `R` which `T` is an algebra over.
For example,
```lean
example : (2:ℤ) • x = (2:ℚ≥0) • x := by module
```
fails since `ℤ` is not a `ℚ≥0`-algebra and `ℚ≥0` is not a `ℤ`-algebra, but
```lean
example : (2:ℤ) • x = (2:ℚ≥0) • x := by module ℚ
```
works since `ℚ` is both a `ℤ`-algebra and a `ℚ≥0`-algebra.
This PR is a quick proof-of-concept implementation, just to record the desired approach and tactic syntax. It should not be merged as-is. It has with a lot of code duplication and should be rewritten more efficiently (for example, `parse` and `parseEnsuringType` should be merged to a single function, and the `some`/`none` cases in `matchScalarsAux` should be merged to a uniform treatment) before being considered for merging to Mathlib.
---
[](https://gitpod.io/from-referrer/)
|
t-meta
merge-conflict
|
158/35 |
Mathlib/Tactic/Module.lean,test/module.lean |
2 |
1 |
['github-actions'] |
nobody |
330-11524 10 months ago |
330-11524 10 months ago |
0-0 0 seconds |
12414 |
adomani author:adomani |
test: lint and unlint `·` |
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict |
64/14 |
Archive/Wiedijk100Theorems/CubingACube.lean,Mathlib/Algebra/Module/Submodule/Bilinear.lean,Mathlib/Tactic/Linter/Multigoal.lean,test/Multigoal.lean |
4 |
4 |
['adomani', 'github-actions', 'grunweg', 'leanprover-bot'] |
nobody |
325-73709 10 months ago |
325-73709 10 months ago |
0-0 0 seconds |
16925 |
YnirPaz author:YnirPaz |
feat(SetTheory/Cardinal/Cofinality): aleph index of singular cardinal has infinite cofinality |
Prove `Ordinal.aleph0_le_cof_of_not_isRegular`.
---
[](https://gitpod.io/from-referrer/)
|
t-set-theory
merge-conflict
WIP
|
6/0 |
Mathlib/SetTheory/Cardinal/Cofinality.lean |
1 |
4 |
['YnirPaz', 'github-actions', 'vihdzp'] |
nobody |
324-45291 10 months ago |
324-45291 10 months ago |
2-57220 2 days |
16647 |
eric-wieser author:eric-wieser |
feat: partitions of lists |
The length of this list is the bell numbers.
---
[](https://gitpod.io/from-referrer/)
|
t-data
t-combinatorics
merge-conflict
|
311/0 |
Mathlib.lean,Mathlib/Data/List/Partition.lean |
2 |
1 |
['github-actions'] |
nobody |
323-7783 10 months ago |
323-7783 10 months ago |
0-0 0 seconds |
9605 |
davikrehalt author:davikrehalt |
feat(Data/Finset & List): Add Lemmas for Sorting and Filtering |
This PR includes several useful lemmas to the Data/Finset and Data/List modules in Lean's mathlib:
1. `toFinset_filter` (List): Shows that filtering commutes with toFinset.
2. `toFinset_is_singleton_implies_replicate` (List): Shows a list with a singleton toFinset is a List.replicate.
3. `filter_sort_commute` (Finset): Sorting and filtering can be interchanged in Finsets.
4. `Sorted.filter` (List): A sorted list stays sorted after filtering.
5. `Sorted.append_largest` (List): Appending the largest element keeps a list sorted.
6. `sort_monotone_map` (Finset): Relates sorting of a Finset after mapping to sorting of a list.
7. `sort_insert_largest` (Finset): Sorting a Finset with an inserted largest element.
8. `sort_range` (Finset): Sorting a range in a Finset equals the corresponding range list.
9. ~~`filter_eval_true` (List): Filtering a list with a predicate always true keeps the list unchanged.~~
10. ~~`filter_eval_false` (List): Filtering with an always-false predicate gives an empty list.~~
11. ~~`pairwise_concat` (List): Iff condition for Pairwise relation in concatenated lists (similar to pairwise_join).~~
12. `list_map_toFinset` (Finset): toFinset commutes with map under injection
---
- [x] depends on: #15952
This is my first PR to mathlib, so I'm not too familiar with etiquette's and more specifically there are two proofs in the PR which uses aesop, and I am not sure if it's frowned upon. I kept the aesop in there for now as I couldn't construct very short proofs otherwise. The sort_range function proof was suggested in https://leanprover.zulipchat.com/#narrow/stream/113489-new-members/topic/Computing.20Finset.20sort.20of.20Finset.20range/near/410346731 by Ruben Van de Velde. Thanks for your time for improving this PR. |
t-data
new-contributor
merge-conflict
please-adopt
awaiting-author
|
71/0 |
Mathlib/Data/Finset/Basic.lean,Mathlib/Data/Finset/Image.lean,Mathlib/Data/Finset/Sort.lean,Mathlib/Data/List/Sort.lean |
4 |
30 |
['YaelDillies', 'davikrehalt', 'eric-wieser', 'github-actions', 'jcommelin', 'leanprover-community-mathlib4-bot', 'urkud', 'vihdzp'] |
YaelDillies assignee:YaelDillies |
317-48478 10 months ago |
344-17269 11 months ago |
12-48560 12 days |
5364 |
thorimur author:thorimur |
feat: `wlog ... replacing` |
This allows hypotheses to be removed from the set of generalized hypotheses. E.g. `wlog h : P replacing h'` will remove `h'` from the hypotheses of the type of `this` and from the context of the goal that will suppose `h`. See [zulip](https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/wlog.20.2E.2E.2E.20replacing.20.2E.2E.2E.3F).
---
[](https://gitpod.io/from-referrer/)
|
t-meta
merge-conflict
|
125/18 |
Mathlib/Tactic/WLOG.lean,test/wlog.lean |
2 |
2 |
['thorimur', 'urkud'] |
nobody |
313-35135 10 months ago |
313-35135 10 months ago |
0-0 0 seconds |
9654 |
urkud author:urkud |
feat: add `@[mk_eq]` version of `@[mk_iff]` |
The new attribute generates theorems like
```lean
List.chain_eq : @List.Chain = fun {α} R a a_1 => a_1 = [] ∨ ∃ b l, R a b ∧ List.Chain R b l ∧ a_1 = b :: l
```
and is useful to rewrite in a theorem that argues about the properties of an unapplied inductive predicate.
---
[](https://gitpod.io/from-referrer/)
|
t-meta
merge-conflict
awaiting-author
|
63/9 |
Mathlib/Lean/Meta.lean,Mathlib/Tactic/MkIffOfInductiveProp.lean,test/MkIffOfInductive.lean |
3 |
6 |
['Vierkantor', 'github-actions', 'urkud'] |
nobody |
313-34889 10 months ago |
313-34889 10 months ago |
25-70815 25 days |
16704 |
AntoineChambert-Loir author:AntoineChambert-Loir |
feat(Mathlib.Data.Ordering.Dickson): Dickson orders |
Dickson orders are a particular class of well founded orders
characterized by the fact that every nonempty set has finitely many minimal elements.
They appear in the classical theory of Groebner bases because it is easier to prove
that some sets are well founded using this property.
WiP. In the `tfae` function, property 2 is exactly `Set.PartiallyWellOrderedOn`, so the PR should be rewritten so as to use that property (and not define `IsDickson`).
---
[](https://gitpod.io/from-referrer/)
|
t-order
merge-conflict
WIP
|
324/0 |
Mathlib.lean,Mathlib/Data/Ordering/Dickson.lean,scripts/noshake.json |
3 |
9 |
['AntoineChambert-Loir', 'b-mehta', 'github-actions'] |
nobody |
313-13446 10 months ago |
313-13446 10 months ago |
2-84515 2 days |
16355 |
Ruben-VandeVelde author:Ruben-VandeVelde |
feat: odd_{add,sub}_one |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-number-theory
merge-conflict
awaiting-author
label:t-algebra$ |
12/0 |
Mathlib/Algebra/Ring/Int.lean,Mathlib/Algebra/Ring/Parity.lean |
2 |
4 |
['Ruben-VandeVelde', 'github-actions', 'urkud'] |
nobody |
312-47643 10 months ago |
312-47643 10 months ago |
0-57608 16 hours |
8479 |
alexjbest author:alexjbest |
feat: use leaff in CI |
[Leaff](https://github.com/alexjbest/leaff) is an experimental lean-diff tool, this PR is to experiment with adding it as a CI step.
---
I'm not sure yet if it is best to have this always run or only run on request (like bench).
If it is always run should it post a comment or simply leave its output it the actions log (maybe as a summary object)
the current iteration runs and updates a sticky comment with the latest result
[](https://gitpod.io/from-referrer/)
|
merge-conflict
awaiting-author
WIP
|
340/0 |
.github/workflows/bors.yml,.github/workflows/build.yml,.github/workflows/build.yml.in,.github/workflows/build_fork.yml |
4 |
11 |
['alexjbest', 'github-actions', 'grunweg', 'kim-em', 'mathlib-bors', 'urkud'] |
nobody |
312-38397 10 months ago |
312-38411 10 months ago |
0-0 0 seconds |
8638 |
alreadydone author:alreadydone |
refactor: noncommutative tensor product |
Co-authored-by: Eric Wieser
Co-authored-by: Jujian Zhang
This draft PR currently only generalizes a single file TensorProduct.lean; it allows TensorProduct to be taken over a non-commutative ring. Most of the declarations in TensorProduct.lean are now generalized to the non-commutative setting, and very few are deleted (their commutative version will be restored in another file).
Next plans:
+ Change the namespace in TensorProduct.lean from TensorProduct to NonCommTensorProduct, and remove the #aligns
+ I plan to use the same notation for the non-commutative and the commutative TensorProduct, and the user will need to `open scoped` different namespaces to use the one of their choice.
+ Start a new file TensorProduct/Comm.lean, copy the content of TensorProduct.lean on master into it, change the definition TensorProduct to be semi-reducibly defeq to NonCommTensorProduct (in order to support more instances or unify non-defeq instances that become prop-eq in the commutative setting, e.g. we've chosen the R-action on a tensor product over commutative R to come from the left factor, since the action from the right factor is the same), and reuse the NonComm constructions as much as possible. We then change all files that imports TensorProduct.lean to import TensorProduct/Comm.lean instead. Once we do that, mathlib would compile and this PR would be complete. We can gradually generalize other files about tensor products this way.
In this PR:
`TensorProduct.map` is now defined in terms of `lTensor` and `rTensor` rather than the other way around, which requires moving `lTensor` and `rTensor` up from their original location. The definition of `rid` also becomes more challenging and is moved down.
An evident observation is that actions on the domain of AddMonoidHom / LinearMap is really natural in the context of tensor products and Hom-tensor adjunction (`TensorProduct.lift`), not the default actions on the codomain. For example, it allows us to write the "balanced biadditive monoid homs" in #8536 as simply `N →ₗ[R] M →+ P` (where the right R-action on M turns into the left action on `M →+ P`).
For this reason, we disable the default instances `AddMonoidHom/LinearMap.module` at the beginning of the file and enable the `AddMonoidHom/LinearMap.domModule` instances instead. (The action on the codomain would be necessary for the non-commutative version of [TensorProduct.lTensorHomToHomLTensor](https://leanprover-community.github.io/mathlib4_docs/Mathlib/LinearAlgebra/TensorProduct.html#TensorProduct.lTensorHomToHomLTensor) (in the form of `P ⊗[R] (M →+ Q) →+ M →+ P ⊗[R] Q`), but I've deleted it for now.)
We register actions on the left factor of a tensor product as the default instance, but we also talk about actions on the right factor (`attribute [local instance] rightModule`).
The Tensor-Hom adjunction #8495 is now `uncurryEquiv` in this PR.
#8519 is now included in this PR and #8584 is now called `lift` in this PR.
`CharacterModule.homEquiv` in #8559 can be obtained by combining `liftEquiv` and `flipMop` in this PR (except for a mop). To refactor the commutative tensor product, we'd need to transfer many R^mop-action to R-action and R^mop-LinearMaps to R-LinearMaps, which can be achieved via `Module.compHom` and `LinearMap.restrictScalars` (requires `LinearMap.CompatibleSMul` instance) given `RingEquiv.toOpposite`. `LinearMap.characterfy` and `CharacterModule.cong` could be obtained from `LinearMap.compAddMonoidHom` in this PR.
TODO:
+ Move delarations that belong to other files.
+ Change docstrings that are no longer accurate.
+ Fix some argument order to be more natural.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
WIP
label:t-algebra$ |
793/676 |
Mathlib/Algebra/Module/LinearMap.lean,Mathlib/GroupTheory/GroupAction/DomAct/Basic.lean,Mathlib/LinearAlgebra/TensorProduct.lean |
3 |
6 |
['alreadydone', 'eric-wieser', 'grhkm21', 'jjaassoonn'] |
nobody |
311-73856 10 months ago |
430-76042 1 year ago |
0-0 0 seconds |
14598 |
Command-Master author:Command-Master |
chore: add typeclasses to unify various `add_top`, `add_eq_top`, etc. |
Add the four typeclasses `IsTopAbsorbing`, `IsBotAbsorbing`, `NoTopSum`, `NoBotSum`, as additive equivalents for `MulZeroClass` and `NoZeroDivisors`. Add instances of these for `ENNReal`, `WithTop α`, `WithBot α`, `PUnit`, `EReal`, `PartENat`, `Measure`, `Interval` and `Filter`.
Also split `Algebra/Order/AddGroupWithTop` to `Algebra/Order/Group/WithTop` and `Algebra/Order/Monoid/WithTop`
---
Previous usages of lemmas with quantified names like `WithTop.add_top` have to be changed to just `add_top`.
`add_lt_top` is `@[simp]`, in accordance with `ENNReal.add_lt_top` being `@[simp]`. This affects `WithTop.add_lt_top` which previously hadn't been `@[simp]`.
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-order
t-algebra
merge-conflict
label:t-algebra$ |
264/195 |
Archive/Wiedijk100Theorems/BallotProblem.lean,Mathlib.lean,Mathlib/Algebra/Order/Group/WithTop.lean,Mathlib/Algebra/Order/GroupWithZero/Canonical.lean,Mathlib/Algebra/Order/Interval/Basic.lean,Mathlib/Algebra/Order/Monoid/Unbundled/Basic.lean,Mathlib/Algebra/Order/Monoid/Unbundled/Defs.lean,Mathlib/Algebra/Order/Monoid/Unbundled/WithTop.lean,Mathlib/Algebra/Order/Monoid/WithTop.lean,Mathlib/Algebra/PUnitInstances/Order.lean,Mathlib/Algebra/Polynomial/Degree/Definitions.lean,Mathlib/Algebra/Polynomial/Monic.lean,Mathlib/Algebra/Tropical/Basic.lean,Mathlib/Analysis/Analytic/Meromorphic.lean,Mathlib/Analysis/Normed/Lp/ProdLp.lean,Mathlib/Analysis/NormedSpace/ENorm.lean,Mathlib/Analysis/SpecialFunctions/JapaneseBracket.lean,Mathlib/Analysis/SpecialFunctions/Log/ENNRealLog.lean,Mathlib/Data/ENNReal/Operations.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/Data/Nat/PartENat.lean,Mathlib/Data/Nat/WithBot.lean,Mathlib/Data/Real/EReal.lean,Mathlib/LinearAlgebra/Lagrange.lean,Mathlib/MeasureTheory/Covering/Differentiation.lean,Mathlib/MeasureTheory/Decomposition/Lebesgue.lean,Mathlib/MeasureTheory/Function/ConditionalExpectation/CondexpL1.lean,Mathlib/MeasureTheory/Function/Jacobian.lean,Mathlib/MeasureTheory/Function/L1Space.lean,Mathlib/MeasureTheory/Function/L2Space.lean,Mathlib/MeasureTheory/Function/LpSeminorm/Basic.lean,Mathlib/MeasureTheory/Function/LpSeminorm/TriangleInequality.lean,Mathlib/MeasureTheory/Function/LpSpace.lean,Mathlib/MeasureTheory/Function/StronglyMeasurable/Basic.lean,Mathlib/MeasureTheory/Function/UniformIntegrable.lean,Mathlib/MeasureTheory/Integral/Bochner.lean,Mathlib/MeasureTheory/Integral/MeanInequalities.lean,Mathlib/MeasureTheory/Integral/SetIntegral.lean,Mathlib/MeasureTheory/Integral/VitaliCaratheodory.lean,Mathlib/MeasureTheory/Measure/Hausdorff.lean,Mathlib/MeasureTheory/Measure/Lebesgue/Basic.lean,Mathlib/MeasureTheory/Measure/LevyProkhorovMetric.lean,Mathlib/MeasureTheory/Measure/MeasureSpace.lean,Mathlib/MeasureTheory/Measure/MeasureSpaceDef.lean,Mathlib/MeasureTheory/Measure/Regular.lean,Mathlib/MeasureTheory/Measure/Typeclasses.lean,Mathlib/NumberTheory/Padics/PadicNumbers.lean,Mathlib/Order/Filter/Pointwise.lean,Mathlib/Probability/Kernel/Defs.lean,Mathlib/Probability/Martingale/Convergence.lean,Mathlib/RingTheory/Multiplicity.lean,Mathlib/RingTheory/MvPowerSeries/NoZeroDivisors.lean,Mathlib/RingTheory/UniqueFactorizationDomain.lean,Mathlib/Topology/EMetricSpace/Defs.lean,Mathlib/Topology/MetricSpace/Bounded.lean,Mathlib/Topology/MetricSpace/HausdorffDistance.lean,Mathlib/Topology/MetricSpace/Lipschitz.lean |
57 |
30 |
['Command-Master', 'YaelDillies', 'github-actions'] |
nobody |
311-19044 10 months ago |
311-19044 10 months ago |
7-45599 7 days |
12778 |
MichaelStollBayreuth author:MichaelStollBayreuth |
perf: decouple algebraic and order hierarchies in type class search |
Based on the experience gained with [#12680](https://github.com/leanprover-community/mathlib4/pull/12680), this attempts to decouple the algebraic and order hierarchies in type class search.
* We lower the priorities of instances like `OrderedSemiring.toSemiring` (which are generated by the `extends` clause with default priority 1000) to 50.
* Additionally, we make the default priority available via `open scoped AlgebraOrderInstances` and use that where appropriate.
**Motivation:** Looking at instance synthesization traces, it appears that when (e.g.) presented with the goal to find a `Semiring` instance, the algorithm frequently goes down a rabbit hole trying and failing to find order instances. This seems to be caused by the presence of instances like `OrderedSemiring.toSemiring` with default priority, which are tried early in the search, but lead nowhere (after a fairly long time). These instances are created by declarations of the form
```lean
class OrderedSemiring (α : Type u) extends Semiring α, OrderedAddCommMonoid α where ...
```
which automatically sets up (among other things) an instance `OrderedSemiring.toSemiring` with default piority. It appears that these instances cannot be removed completely (only locally in a module), so the next best solution is to make them low priority (which is possible also for downstream modules). To provide for situations where these instances are desired, we put a default priority version in the scope `AlgebraOrderInstances`.
---
[](https://gitpod.io/from-referrer/)
|
slow-typeclass-synthesis
t-order
t-algebra
merge-conflict
label:t-algebra$ |
306/27 |
Mathlib/Algebra/Algebra/Subalgebra/Order.lean,Mathlib/Algebra/ContinuedFractions/Computation/ApproximationCorollaries.lean,Mathlib/Algebra/ContinuedFractions/Computation/Approximations.lean,Mathlib/Algebra/Module/Rat.lean,Mathlib/Algebra/Module/Submodule/Order.lean,Mathlib/Algebra/Order/AbsoluteValue.lean,Mathlib/Algebra/Order/Algebra.lean,Mathlib/Algebra/Order/Antidiag/Prod.lean,Mathlib/Algebra/Order/Archimedean/Basic.lean,Mathlib/Algebra/Order/BigOperators/Group/Finset.lean,Mathlib/Algebra/Order/BigOperators/Group/List.lean,Mathlib/Algebra/Order/BigOperators/Group/Multiset.lean,Mathlib/Algebra/Order/BigOperators/Ring/Finset.lean,Mathlib/Algebra/Order/BigOperators/Ring/List.lean,Mathlib/Algebra/Order/BigOperators/Ring/Multiset.lean,Mathlib/Algebra/Order/CauSeq/Basic.lean,Mathlib/Algebra/Order/Chebyshev.lean,Mathlib/Algebra/Order/CompleteField.lean,Mathlib/Algebra/Order/Field/Basic.lean,Mathlib/Algebra/Order/Field/Defs.lean,Mathlib/Algebra/Order/Field/Pi.lean,Mathlib/Algebra/Order/Floor.lean,Mathlib/Algebra/Order/Floor/Div.lean,Mathlib/Algebra/Order/Group/Defs.lean,Mathlib/Algebra/Order/Group/Units.lean,Mathlib/Algebra/Order/GroupWithZero/Canonical.lean,Mathlib/Algebra/Order/Hom/Basic.lean,Mathlib/Algebra/Order/Hom/Monoid.lean,Mathlib/Algebra/Order/Interval/Basic.lean,Mathlib/Algebra/Order/Interval/Set/Instances.lean,Mathlib/Algebra/Order/Invertible.lean,Mathlib/Algebra/Order/Kleene.lean,Mathlib/Algebra/Order/Module/Algebra.lean,Mathlib/Algebra/Order/Module/Defs.lean,Mathlib/Algebra/Order/Module/Pointwise.lean,Mathlib/Algebra/Order/Monoid/Basic.lean,Mathlib/Algebra/Order/Monoid/Canonical/Defs.lean,Mathlib/Algebra/Order/Monoid/Defs.lean,Mathlib/Algebra/Order/Monoid/OrderDual.lean,Mathlib/Algebra/Order/Monoid/Prod.lean,Mathlib/Algebra/Order/Nonneg/Field.lean,Mathlib/Algebra/Order/Nonneg/Ring.lean,Mathlib/Algebra/Order/Pi.lean,Mathlib/Algebra/Order/Positive/Field.lean,Mathlib/Algebra/Order/Positive/Ring.lean,Mathlib/Algebra/Order/Rearrangement.lean,Mathlib/Algebra/Order/Ring/Basic.lean,Mathlib/Algebra/Order/Ring/Defs.lean,Mathlib/Algebra/Order/Ring/InjSurj.lean,Mathlib/Algebra/Order/Ring/Pow.lean,Mathlib/Algebra/Order/Sub/WithTop.lean,Mathlib/Algebra/Order/ToIntervalMod.lean,Mathlib/Algebra/Ring/BooleanRing.lean,Mathlib/AlgebraicGeometry/Morphisms/RingHomProperties.lean,Mathlib/AlgebraicTopology/FundamentalGroupoid/Basic.lean,Mathlib/Analysis/BoundedVariation.lean,Mathlib/Analysis/Complex/UpperHalfPlane/Metric.lean,Mathlib/Analysis/Convex/Basic.lean,Mathlib/Analysis/Convex/Cone/Basic.lean,Mathlib/Analysis/Convex/Cone/Closure.lean,Mathlib/Analysis/Convex/Cone/Pointed.lean,Mathlib/Analysis/Convex/Cone/Proper.lean,Mathlib/Analysis/Convex/Exposed.lean,Mathlib/Analysis/Convex/Extrema.lean,Mathlib/Analysis/Convex/Function.lean,Mathlib/Analysis/Convex/Gauge.lean,Mathlib/Analysis/Convex/GaugeRescale.lean,Mathlib/Analysis/Convex/Hull.lean,Mathlib/Analysis/Convex/Join.lean,Mathlib/Analysis/Convex/Mul.lean,Mathlib/Analysis/Convex/Quasiconvex.lean,Mathlib/Analysis/Convex/SpecificFunctions/Pow.lean,Mathlib/Analysis/Convex/Star.lean,Mathlib/Analysis/Convex/Strict.lean,Mathlib/Analysis/InnerProductSpace/Orientation.lean,Mathlib/Analysis/MeanInequalities.lean,Mathlib/Analysis/SpecialFunctions/Gamma/BohrMollerup.lean,Mathlib/Analysis/SpecialFunctions/Polynomials.lean,Mathlib/Analysis/SpecificLimits/FloorPow.lean,Mathlib/Analysis/SpecificLimits/Normed.lean,Mathlib/Combinatorics/Optimization/ValuedCSP.lean,Mathlib/Combinatorics/Pigeonhole.lean,Mathlib/Combinatorics/SetFamily/FourFunctions.lean,Mathlib/Data/DFinsupp/Lex.lean,Mathlib/Data/DFinsupp/Multiset.lean,Mathlib/Data/DFinsupp/Order.lean,Mathlib/Data/Finset/MulAntidiagonal.lean,Mathlib/Data/Finsupp/Lex.lean,Mathlib/Data/Finsupp/Multiset.lean,Mathlib/Data/Finsupp/Order.lean,Mathlib/Data/Int/Log.lean,Mathlib/Data/Multiset/Antidiagonal.lean,Mathlib/Data/Multiset/Basic.lean,Mathlib/Data/Multiset/Bind.lean,Mathlib/Data/Nat/Cast/Field.lean,Mathlib/Data/Nat/Cast/Order/Basic.lean,Mathlib/Data/Nat/Choose/Bounds.lean,Mathlib/Data/PNat/Factors.lean,Mathlib/Data/Rat/Denumerable.lean,Mathlib/Data/Set/Pointwise/Interval.lean |
135 |
34 |
['MichaelStollBayreuth', 'YaelDillies', 'github-actions', 'leanprover-bot'] |
nobody |
311-17947 10 months ago |
311-17947 10 months ago |
18-19513 18 days |
18636 |
adomani author:adomani |
Test/latest import report dev |
This PR is a test accompanying #18631.
---
[](https://gitpod.io/from-referrer/)
|
CI
merge-conflict
|
147/0 |
.github/workflows/latest_import.yml,lakefile.lean |
2 |
1 |
['github-actions'] |
nobody |
310-6315 10 months ago |
310-6315 10 months ago |
0-0 0 seconds |
16885 |
metinersin author:metinersin |
feat(ModelTheory/Complexity): define literals |
Defines `FirstOrder.Language.BoundedFormula.IsLiteral` and `FirstOrder.Language.BoundedFormula.simpleNot` - an auxiliary operation that takes the negation of a formula and does some simplification.
---
- [x] depends on: #16800
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-logic
merge-conflict
awaiting-author
|
148/5 |
Mathlib/ModelTheory/Complexity.lean,Mathlib/ModelTheory/Equivalence.lean,Mathlib/ModelTheory/Semantics.lean,Mathlib/ModelTheory/Syntax.lean |
4 |
20 |
['YaelDillies', 'awainverse', 'github-actions', 'mathlib4-dependent-issues-bot', 'metinersin'] |
nobody |
308-61565 10 months ago |
308-61565 10 months ago |
0-19926 5 hours |
9341 |
winstonyin author:winstonyin |
feat: Naturality of integral curves |
Let `v` and `v'` be sections of the tangent bundle of manifolds `M` and `M'`, respectively, and let `f : M → M'` be a differentiable map. Then `f` maps integral curves of `v` to integral curves of `v'` if and only if `v` and `v'` are `f`-related.
- [x] depends on: #8483
---
[](https://gitpod.io/from-referrer/)
|
t-differential-geometry
merge-conflict
awaiting-author
|
45/0 |
Mathlib/Geometry/Manifold/IntegralCurve.lean,Mathlib/Topology/Algebra/Module/Basic.lean |
2 |
n/a |
['github-actions', 'grunweg', 'leanprover-community-mathlib4-bot', 'winstonyin'] |
nobody |
305-26988 10 months ago |
unknown |
unknown |
13248 |
hcWang942 author:hcWang942 |
feat: basic concepts of auction theory |
## Description
Formalise some core concepts and results in auction theory: this includes definitions for first-price and second-price auctions, as well as several fundamental results and helping lemmas.
This is the very first PR of the project formalizing core concepts and results in auction theory.
Our group is working on more contributions on the formalization of game theory prefix.
Co-authored-by: Ma Jiajun
## Reference
Roughgarden, Tim. ***Twenty Lectures on Algorithmic Game Theory***. Cambridge University Press, 2020. [Link](https://www.cambridge.org/core/books/twenty-lectures-on-algorithmic-game-theory/A9D9427C8F43E7DAEF8C702755B6D72B)
---
- [x] Will depend on #14163 once that PR is merged. The Fintype lemmas introduced by this PR have been added in that PR and will be removed from here once that PR gets merged
## Current plan for formalization of Game Theory
The current plan for the formalizing of Game Theory include:
#### 1. Auction Theory. 🎉 _(200+ lines, this PR)_
- Essential definitions of Sealed-bid auction, First-price auction and Second-price auction.
- First-price auction has no dominant strategy.
- Second-price auction has dominant strategy. (Second-price auction is DSIC)
#### 2. Mechanism design & Myerson's Lemma. 🎉 (400+ lines, pending for modification to Mathlib Standard)
- Mechanism design
An allocation rule is implementable if there exists
- Dominant Strategy Incentive Compatible (DSIC) payment rule
- An allocation rule is monotone if for every bidder’s gain is nondecreasing w.r.t. her/his bid
- Myerson's Lemma
Implementable ⇔ Monotone
In the above case, the DSIC payment rule is unique.
#### 3. von Neumann‘s Minimax Theorem. 🎉 (800+ lines, pending for modification to Mathlib Standard)
- Equilibrium in zero sum game
- Formalization strategy: via Loomis’s theorem.
#### 4. Nash Equilibrium. 🎉 (pending for modification to Mathlib Standard)
#### 5. Brouwer fixed-point theorem. (Work in Progress)
#### 6. More Mechanism design. (Planning)
|
new-contributor
t-logic
merge-conflict
awaiting-author
|
204/0 |
Mathlib.lean,Mathlib/GameTheory/Auction/Basic.lean,docs/references.bib |
3 |
148 |
['Shreyas4991', 'YaelDillies', 'eric-wieser', 'faenuccio', 'github-actions', 'grunweg', 'hcWang942', 'tb65536', 'urkud', 'vihdzp'] |
hcWang942 assignee:hcWang942 |
304-13997 10 months ago |
unknown |
unknown |
17675 |
FR-vdash-bot author:FR-vdash-bot |
perf: do not search algebraic hierarchy when searching `FunLike` hierarchy |
---
Unification is still very slow.
[](https://gitpod.io/from-referrer/)
|
slow-typeclass-synthesis
t-algebra
merge-conflict
label:t-algebra$ |
144/4 |
Mathlib.lean,Mathlib/Algebra/Algebra/Equiv.lean,Mathlib/Algebra/Algebra/Hom.lean,Mathlib/Algebra/Algebra/NonUnitalHom.lean,Mathlib/Algebra/Algebra/Rat.lean,Mathlib/Algebra/Group/Equiv/Basic.lean,Mathlib/Algebra/GroupWithZero/Hom.lean,Mathlib/Algebra/Module/Equiv/Defs.lean,Mathlib/Algebra/Module/LinearMap/Defs.lean,Mathlib/Algebra/Order/Hom/Basic.lean,Mathlib/Algebra/Ring/CentroidHom.lean,Mathlib/Algebra/Ring/Equiv.lean,Mathlib/Algebra/Ring/Hom/Defs.lean,Mathlib/Algebra/Star/StarAlgHom.lean,Mathlib/Analysis/Normed/Algebra/Spectrum.lean,Mathlib/Analysis/Normed/Operator/LinearIsometry.lean,Mathlib/GroupTheory/GroupAction/Hom.lean,Mathlib/RingTheory/Bialgebra/Equiv.lean,Mathlib/RingTheory/Bialgebra/Hom.lean,Mathlib/RingTheory/Coalgebra/Equiv.lean,Mathlib/Topology/Algebra/Module/Basic.lean,Mathlib/Util/SetSynthOrder.lean,MathlibTest/TCSynth.lean,scripts/noshake.json |
24 |
5 |
['FR-vdash-bot', 'github-actions', 'leanprover-bot'] |
nobody |
303-75530 9 months ago |
303-75530 9 months ago |
0-0 0 seconds |
9344 |
erdOne author:erdOne |
feat: Add `AddGroup.FG` -> `Module.Finite ℤ` as instances |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
awaiting-author
label:t-algebra$ |
4/0 |
Mathlib/RingTheory/Finiteness.lean |
1 |
4 |
['alreadydone', 'erdOne', 'leanprover-bot'] |
nobody |
302-84790 9 months ago |
302-84790 9 months ago |
0-0 0 seconds |
12133 |
ADedecker author:ADedecker |
feat: generalize instIsLowerProd to arbitrary products |
Also change a bit the proof of the product case to match my own taste, feel free to tell if you prefer the old one.
---
[](https://gitpod.io/from-referrer/)
|
t-order
t-topology
merge-conflict
awaiting-author
|
34/14 |
Mathlib/Topology/Constructions.lean,Mathlib/Topology/Order/LowerUpperTopology.lean |
2 |
13 |
['Ruben-VandeVelde', 'TwoFX', 'github-actions', 'jcommelin', 'mans0954', 'mathlib-bors', 'riccardobrasca'] |
nobody |
302-8144 9 months ago |
302-8144 9 months ago |
63-69206 63 days |
16637 |
FR-vdash-bot author:FR-vdash-bot |
perf: reorder `extends` of `(Add)Monoid` |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
WIP
label:t-algebra$ |
46/51 |
Mathlib/Algebra/Algebra/Hom.lean,Mathlib/Algebra/BigOperators/Ring/List.lean,Mathlib/Algebra/GCDMonoid/Basic.lean,Mathlib/Algebra/Group/Defs.lean,Mathlib/Algebra/Group/Ext.lean,Mathlib/Algebra/Group/Opposite.lean,Mathlib/Algebra/Group/Prod.lean,Mathlib/Algebra/Order/Group/Unbundled/Abs.lean,Mathlib/Algebra/Polynomial/Roots.lean,Mathlib/Algebra/Ring/SumsOfSquares.lean,Mathlib/CategoryTheory/Preadditive/FunctorCategory.lean,Mathlib/Data/Finset/NoncommProd.lean,Mathlib/GroupTheory/Congruence/Defs.lean,Mathlib/GroupTheory/Torsion.lean,Mathlib/LinearAlgebra/LinearPMap.lean,Mathlib/LinearAlgebra/TensorProduct/Basic.lean,Mathlib/Order/Filter/Germ/Basic.lean,Mathlib/RingTheory/Bialgebra/Hom.lean,Mathlib/RingTheory/Coalgebra/Hom.lean,Mathlib/RingTheory/TensorProduct/MvPolynomial.lean |
20 |
3 |
['FR-vdash-bot', 'github-actions', 'leanprover-bot'] |
nobody |
302-7382 9 months ago |
302-7382 9 months ago |
1-49655 1 day |
18765 |
FR-vdash-bot author:FR-vdash-bot |
chore: changing `outParam` of `MulActionSemiHomClass` |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
label:t-algebra$ |
60/34 |
Mathlib/Algebra/Algebra/NonUnitalHom.lean,Mathlib/Algebra/Category/ModuleCat/Limits.lean,Mathlib/Algebra/Module/LinearMap/Defs.lean,Mathlib/GroupTheory/GroupAction/Hom.lean |
4 |
4 |
['FR-vdash-bot', 'github-actions', 'leanprover-bot'] |
nobody |
301-50043 9 months ago |
301-50043 9 months ago |
0-0 0 seconds |
14739 |
urkud author:urkud |
feat(Measure): add `gcongr` lemmas |
---
[](https://gitpod.io/from-referrer/) |
t-measure-probability
merge-conflict
awaiting-author
WIP
help-wanted
|
12/8 |
Mathlib/MeasureTheory/Covering/Differentiation.lean,Mathlib/MeasureTheory/Function/SimpleFunc.lean,Mathlib/MeasureTheory/Integral/SetToL1.lean,Mathlib/MeasureTheory/Measure/MeasureSpace.lean,Mathlib/Probability/Kernel/Disintegration/Density.lean |
5 |
3 |
['github-actions', 'kim-em', 'urkud'] |
nobody |
301-7078 9 months ago |
301-7078 9 months ago |
0-66587 18 hours |
15822 |
kmill author:kmill |
feat: greedy colorings of finite graphs |
Proves that the greedy coloring only takes `G.maxDegree + 1` colors.
---
[](https://gitpod.io/from-referrer/)
|
t-combinatorics
merge-conflict
|
159/0 |
Mathlib/Combinatorics/SimpleGraph/ConcreteColorings.lean |
1 |
1 |
['github-actions'] |
nobody |
298-75236 9 months ago |
298-75236 9 months ago |
0-0 0 seconds |
8661 |
joelriou author:joelriou |
feat(CategoryTheory/Sites): descent of sheaves |
In this PR, it is shown that the category of sheaves on a site `(C, J)` identifies as a full subcategory of a category of families of sheaves equipped with a descent data (for a family of objects which cover the final object). Under suitable conditions, it shall be shown that this is an equivalence of categories (TODO).
---
This shall be split in small PRs later.
- [x] depends on: #8622
- [x] depends on: #8632
[](https://gitpod.io/from-referrer/)
|
t-category-theory
merge-conflict
WIP
|
1396/26 |
Mathlib.lean,Mathlib/CategoryTheory/Over.lean,Mathlib/CategoryTheory/Sites/CoverPreserving.lean,Mathlib/CategoryTheory/Sites/Descent.lean,Mathlib/CategoryTheory/Sites/EqualizerSheafCondition.lean,Mathlib/CategoryTheory/Sites/InducedTopology.lean,Mathlib/CategoryTheory/Sites/ObjectsCoverTop.lean,Mathlib/CategoryTheory/Sites/Over.lean,Mathlib/CategoryTheory/Sites/SheafHom.lean,Mathlib/CategoryTheory/Sites/Sieves.lean |
10 |
3 |
['github-actions', 'leanprover-community-mathlib4-bot'] |
nobody |
298-70764 9 months ago |
592-6837 1 year ago |
0-0 0 seconds |
19055 |
JLimperg author:JLimperg |
Test precompilation (batteries + aesop) again |
|
merge-conflict |
9/8 |
lake-manifest.json,lakefile.lean |
2 |
5 |
['JLimperg', 'github-actions', 'leanprover-bot'] |
nobody |
298-52407 9 months ago |
298-52407 9 months ago |
0-0 0 seconds |
10476 |
shuxuezhuyi author:shuxuezhuyi |
feat(Topology/UniformSpace): define uniform preordered space |
We define the semi-uniform structure and the uniform preordered space.
---
[](https://gitpod.io/from-referrer/)
|
t-topology
merge-conflict
awaiting-author
|
94/0 |
Mathlib.lean,Mathlib/Topology/UniformSpace/UniformOrder.lean,docs/references.bib |
3 |
2 |
['shuxuezhuyi'] |
nobody |
297-57418 9 months ago |
297-57418 9 months ago |
10-33091 10 days |
17623 |
FR-vdash-bot author:FR-vdash-bot |
feat(Algebra/Order/GroupWithZero/Unbundled): add some lemmas |
Some lemmas in `Algebra.Order.GroupWithZero.Unbundled` have incorrect or unsatisfactory names, or assumptions that can be omitted using `ZeroLEOneClass`. The lemmas added in this PR are versions of existing lemmas that use the correct or better name or `ZeroLEOneClass` to omit an assumption. The original lemmas will be deprecated in #17593.
| New name | Old name |
|-------------------------|-------------------------|
| `mul_le_one_left₀` | `Left.mul_le_one_of_le_of_le` |
| `mul_lt_one_of_le_of_lt_left₀` (`0 ≤ ·` version) / `mul_lt_one_of_le_of_lt_of_pos_left` | `Left.mul_lt_of_le_of_lt_one_of_pos` |
| `mul_lt_one_of_lt_of_le_left₀` | `Left.mul_lt_of_lt_of_le_one_of_nonneg` |
| `mul_le_one_right₀` | `Right.mul_le_one_of_le_of_le` |
| `mul_lt_one_of_lt_of_le_right₀` (`0 ≤ ·` version) / `mul_lt_one_of_lt_of_le_of_pos_right` | `Right.mul_lt_one_of_lt_of_le_of_pos` |
| `mul_lt_one_of_le_of_lt_right₀` | `Right.mul_lt_one_of_le_of_lt_of_nonneg` |
The following lemmas use `ZeroLEOneClass`.
| New name | Old name |
|-------------------------|-------------------------|
| `(Left.)one_le_mul₀` | `Left.one_le_mul_of_le_of_le` |
| `Left.one_lt_mul_of_le_of_lt₀` | `Left.one_lt_mul_of_le_of_lt_of_pos` |
| `Left.one_lt_mul_of_lt_of_le₀` | `Left.lt_mul_of_lt_of_one_le_of_nonneg` / `one_lt_mul_of_lt_of_le` (still there) |
| `(Left.)one_lt_mul₀` | |
| `Right.one_le_mul₀` | `Right.one_le_mul_of_le_of_le` |
| `Right.one_lt_mul_of_lt_of_le₀` | `Right.one_lt_mul_of_lt_of_le_of_pos` |
| `Right.one_lt_mul_of_le_of_lt₀` | `Right.one_lt_mul_of_le_of_lt_of_nonneg` / `one_lt_mul_of_le_of_lt` (still there) / `one_lt_mul` (still there) |
| `Right.one_lt_mul₀` | `Right.one_lt_mul_of_lt_of_lt` |
---
Split from #17593.
[](https://gitpod.io/from-referrer/)
|
awaiting-zulip
t-order
t-algebra
merge-conflict
label:t-algebra$ |
146/44 |
Mathlib/Algebra/Order/GroupWithZero/Canonical.lean,Mathlib/Algebra/Order/GroupWithZero/Unbundled.lean |
2 |
11 |
['FR-vdash-bot', 'YaelDillies', 'github-actions', 'j-loreaux'] |
nobody |
296-80760 9 months ago |
296-80760 9 months ago |
33-64877 33 days |
18969 |
alreadydone author:alreadydone |
chore: generalize Module to NonUnitalSemiring |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
WIP
label:t-algebra$ |
94/75 |
Mathlib/Algebra/Category/ModuleCat/Presheaf.lean,Mathlib/Algebra/Group/Action/Defs.lean,Mathlib/Algebra/Group/Action/End.lean,Mathlib/Algebra/Group/Action/Prod.lean,Mathlib/Algebra/Group/Action/TypeTags.lean,Mathlib/Algebra/GroupWithZero/Action/Defs.lean,Mathlib/Algebra/Module/Defs.lean,Mathlib/Algebra/Module/Submodule/Defs.lean,Mathlib/Algebra/Polynomial/Div.lean,Mathlib/Algebra/Polynomial/Laurent.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Group.lean,Mathlib/AlgebraicGeometry/Limits.lean,Mathlib/AlgebraicGeometry/ProjectiveSpectrum/Scheme.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Order.lean,Mathlib/Analysis/Distribution/SchwartzSpace.lean,Mathlib/Geometry/Manifold/Instances/Sphere.lean,Mathlib/GroupTheory/CoprodI.lean,Mathlib/LinearAlgebra/FreeModule/IdealQuotient.lean,Mathlib/LinearAlgebra/LinearDisjoint.lean,Mathlib/LinearAlgebra/Matrix/SesquilinearForm.lean,Mathlib/LinearAlgebra/TensorProduct/Submodule.lean,Mathlib/RingTheory/Filtration.lean,Mathlib/RingTheory/Flat/FaithfullyFlat.lean,Mathlib/RingTheory/Ideal/Cotangent.lean,Mathlib/RingTheory/Ideal/Defs.lean,Mathlib/RingTheory/Ideal/Lattice.lean,Mathlib/RingTheory/Ideal/Operations.lean,Mathlib/RingTheory/Ideal/Prod.lean,Mathlib/RingTheory/Presentation.lean,Mathlib/RingTheory/Smooth/Kaehler.lean,Mathlib/RingTheory/TensorProduct/MvPolynomial.lean |
31 |
11 |
['alreadydone', 'eric-wieser', 'github-actions', 'leanprover-bot'] |
nobody |
295-18012 9 months ago |
295-18012 9 months ago |
0-0 0 seconds |
16361 |
vihdzp author:vihdzp |
chore(SetTheory/Ordinal/FixedPointApproximants): golf + better variable management |
We avoid making `f : α →o α` and `x : α` explicit arguments when not needed. We then golf most theorems in the file.
---
[](https://gitpod.io/from-referrer/)
|
t-set-theory
t-logic
merge-conflict
awaiting-author
|
68/101 |
Mathlib/SetTheory/Ordinal/FixedPointApproximants.lean |
1 |
8 |
['PhoenixIra', 'YaelDillies', 'github-actions'] |
nobody |
294-13754 9 months ago |
294-13754 9 months ago |
50-29942 50 days |
17513 |
FR-vdash-bot author:FR-vdash-bot |
perf: do not search algebraic hierarchies when using `map_*` lemmas |
---
[](https://gitpod.io/from-referrer/)
|
awaiting-bench
t-algebra
merge-conflict
WIP
label:t-algebra$ |
5/3 |
Mathlib/Algebra/Group/Hom/Defs.lean,Mathlib/GroupTheory/GroupAction/Hom.lean |
2 |
10 |
['FR-vdash-bot', 'github-actions', 'grunweg', 'leanprover-bot'] |
nobody |
291-76954 9 months ago |
291-76954 9 months ago |
4-72589 4 days |
19212 |
Julian author:Julian |
feat(LinearAlgebra): add a variable_alias for VectorSpace |
Taken directly from the variable_alias docs.
Zulip: https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/why.20.5Bvariable_alias.5D.20attribute.20is.20not.20used.20in.20Mathlib.3F
---
This is the first actual variable alias added to mathlib. I haven't reviewed variable_alias fully, but it seems like there's at least 3 ways they could be distributed in Mathlib:
* alongside whatever subfolder they "belong to" (which is what I've tentatively done here)
* In a file called `Aliases` somewhere near the thing they alias (which seems less discoverable to me)
* In a single file, a la `Mathlib.TrainingWheels` (with some less playful name) which is meant to define a bunch of more "friendly" aliases all in one place.
I kind of like the idea of the third thing as a future module but perhaps it can be synthesized if/when there are more aliases? For now as I say I've done the first one, but please let me know if someone prefers something else.
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
label:t-algebra$ |
25/0 |
Mathlib.lean,Mathlib/LinearAlgebra/VectorSpace.lean,scripts/noshake.json |
3 |
10 |
['Julian', 'PieterCuijpers', 'github-actions', 'urkud'] |
nobody |
290-82199 9 months ago |
290-82199 9 months ago |
7-68492 7 days |
19337 |
zeramorphic author:zeramorphic |
feat(Data/Finsupp): generalise `Finsupp` to any "zero" value |
Remove the explicit dependence of `Finsupp` on `[Zero M]`, instead defining `Finsupp'` (better name pending) to be functions that are equal to a fixed value `z : M` cofinitely often.
This PR is intended to do the initial work of replacing the definition of `Finsupp` with an instantiation of the more general definition, without adding any appropriate API. If accepted, the API development will follow in later PRs.
Issues to consider:
- Naming of `Finsupp'.`
- Where should `Finsupp'` lemmas go? Do they need their own file/folder under `Data/`?
Relevant Zulip threads:
- https://leanprover.zulipchat.com/#narrow/channel/217875-Is-there-code-for-X.3F/topic/Finsupp.20generalisations
- https://leanprover.zulipchat.com/#narrow/channel/217875-Is-there-code-for-X.3F/topic/Finsupp-like.20partial.20function
Comments are welcome.
---
[](https://gitpod.io/from-referrer/)
|
t-data
merge-conflict
|
203/83 |
Archive/Wiedijk100Theorems/Partition.lean,Mathlib/Algebra/MvPolynomial/Basic.lean,Mathlib/Algebra/MvPolynomial/Rename.lean,Mathlib/Algebra/MvPolynomial/Variables.lean,Mathlib/Algebra/Polynomial/Basic.lean,Mathlib/Algebra/Polynomial/Laurent.lean,Mathlib/Data/Finsupp/BigOperators.lean,Mathlib/Data/Finsupp/Defs.lean,Mathlib/Data/Finsupp/Order.lean,Mathlib/Data/Nat/Choose/Multinomial.lean,Mathlib/RingTheory/MvPolynomial/Symmetric/Defs.lean,Mathlib/RingTheory/PowerBasis.lean,scripts/nolints_prime_decls.txt |
13 |
5 |
['github-actions', 'vihdzp', 'zeramorphic'] |
nobody |
288-58276 9 months ago |
288-58276 9 months ago |
4-60621 4 days |
19420 |
vihdzp author:vihdzp |
feat: AM-HM inequality |
We prove the weighted and unweighted AM-HM inequalities in linearly ordered semifields.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
awaiting-author
WIP
label:t-algebra$ |
36/2 |
Mathlib/Algebra/Order/BigOperators/Ring/Finset.lean,Mathlib/Analysis/MeanInequalities.lean |
2 |
7 |
['YaelDillies', 'github-actions', 'vihdzp'] |
nobody |
285-27276 9 months ago |
285-27276 9 months ago |
0-46682 12 hours |
10332 |
adri326 author:adri326 |
feat(Topology/Sets): define regular open sets and their boolean algebra |
Introduces a new module, `Mathlib.Topology.Sets.RegularOpens`, which defines the `IsRegularOpen s` predicate (`interior (closure s) = s`) and `TopologicalSpace.RegularOpens`, the type of bundled regular open sets (defined as `Heyting.Regular (Opens X)`).
A few properties of regular open sets (bundled and unbundled) and `interior (closure s)` are proven,
and a pointwise instance of `MulAction` is provided for regular open sets.
---
This PR belongs to my series of PRs around my formalization of Rubin's theorem.
There are two possible ways to implement `RegularOpens`:
- either construct them by hand and show that they form a boolean algebra (better def-eq but more boilerplate code required)
- or use `Heyting.Regular` on the heyting algebra of `Opens` inherited from the `Frame` instance on them
I first chose to use the former approach, but using the latter cuts the length of the construction of the boolean algebra of regular open sets by 100 lines of code, and allows us to inherit all of the helper lemmas defined for `Heyting.Regular`.
The big downside, though, is that an element of `RegularOpens` isn't defined as a bundled regular open set anymore, but rather as an `Opens` set `s` for which `Opens.interior ↑(Opens.interior ↑sᶜ)ᶜ = s`, so I added an alternative constructor `RegularOpens.of` that instead accepts any set `s` for which `IsRegularOpen s` holds.
Another minor downside is that coercion to a set takes two coercions instead of one.
[](https://gitpod.io/from-referrer/)
|
t-topology
merge-conflict
WIP
|
434/0 |
Mathlib.lean,Mathlib/Data/Set/Pointwise/SMul.lean,Mathlib/Topology/Sets/Opens.lean,Mathlib/Topology/Sets/RegularOpens.lean,docs/references.bib |
5 |
1 |
['adri326'] |
YaelDillies assignee:YaelDillies |
284-85623 9 months ago |
393-84813 1 year ago |
0-0 0 seconds |
14501 |
jjaassoonn author:jjaassoonn |
feat: module structure of filtered colimit of abelian groups over filtered colimit of rings |
This helps defining the module structure of stalks
This contribution was inspired by the AIM workshop "Formalizing algebraic geometry" in June 2024.
---
- [x] depends on: #15315 [I am going to move the result in the new file]
[](https://gitpod.io/from-referrer/)
|
workshop-AIM-AG-2024
t-algebra
t-category-theory
merge-conflict
awaiting-author
label:t-algebra$ |
439/2 |
Mathlib/CategoryTheory/Limits/ConcreteCategory/Basic.lean,Mathlib/CategoryTheory/Limits/ConcreteCategory/WithAlgebraicStructures.lean |
2 |
48 |
['YaelDillies', 'adamtopaz', 'erdOne', 'github-actions', 'jjaassoonn', 'joelriou', 'kbuzzard', 'leanprover-community-mathlib4-bot'] |
joelriou assignee:joelriou |
282-2881 9 months ago |
282-2881 9 months ago |
64-29952 64 days |
18756 |
astrainfinita author:astrainfinita |
refactor: deprecate `DistribMulActionSemiHomClass` `MulSemiringActionSemiHomClass` |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
label:t-algebra$ |
50/28 |
Mathlib/Algebra/Algebra/NonUnitalHom.lean,Mathlib/Algebra/Module/LinearMap/Defs.lean,Mathlib/GroupTheory/GroupAction/Hom.lean |
3 |
4 |
['astrainfinita', 'github-actions', 'leanprover-bot'] |
nobody |
277-23945 9 months ago |
277-23945 9 months ago |
31-75259 31 days |
17071 |
ScottCarnahan author:ScottCarnahan |
feat : (LinearAlgebra/RootSystem) : Separation, base, cartanMatrix |
This PR defines an abstract separation structure for roots, together with the associated base and Cartan Matrix. In general, the good properties will follow from additional order hypotheses on the base ring (implemented in a future PR).
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
WIP
label:t-algebra$ |
111/0 |
Mathlib.lean,Mathlib/LinearAlgebra/RootSystem/Separation.lean |
2 |
1 |
['github-actions'] |
nobody |
277-13846 9 months ago |
277-13846 9 months ago |
20-56416 20 days |
19125 |
yhtq author:yhtq |
feat: add theorems to transfer `IsGalois` between pairs of fraction rings |
feat: add theorems to transfer `IsGalois` between pairs of fraction rings.
- [x] depends on: #18404
- [x] depends on: #19124
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-algebra
merge-conflict
label:t-algebra$ |
121/0 |
Mathlib.lean,Mathlib/FieldTheory/Galois/IsFractionRing.lean,Mathlib/RingTheory/Localization/FractionRing.lean |
3 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'tb65536'] |
nobody |
274-36414 9 months ago |
280-71837 9 months ago |
0-4534 1 hour |
18841 |
hrmacbeth author:hrmacbeth |
chore: change some `linarith`s to `linear_combination`s |
Change 100 `linarith`s to `linear_combination`s; this is generally a slight speedup.
---
[](https://gitpod.io/from-referrer/)
- [x] depends on: #18714 (not strictly blocked by this, but the speed comparison will be more informative after it)
|
merge-conflict
WIP
|
106/107 |
Archive/Imo/Imo1959Q2.lean,Archive/Imo/Imo1988Q6.lean,Archive/Imo/Imo2005Q3.lean,Archive/Imo/Imo2008Q2.lean,Archive/Imo/Imo2008Q3.lean,Archive/Imo/Imo2013Q5.lean,Archive/Imo/Imo2021Q1.lean,Mathlib/Analysis/Analytic/Basic.lean,Mathlib/Analysis/Analytic/Inverse.lean,Mathlib/Analysis/Calculus/BumpFunction/FiniteDimension.lean,Mathlib/Analysis/Complex/AbelLimit.lean,Mathlib/Analysis/Convex/Gauge.lean,Mathlib/Analysis/Convex/Slope.lean,Mathlib/Analysis/Convex/SpecificFunctions/Basic.lean,Mathlib/Analysis/Convex/Uniform.lean,Mathlib/Analysis/Convex/Visible.lean,Mathlib/Analysis/FunctionalSpaces/SobolevInequality.lean,Mathlib/Analysis/Normed/Module/FiniteDimension.lean,Mathlib/Analysis/PSeries.lean,Mathlib/Analysis/SpecialFunctions/Gamma/BohrMollerup.lean,Mathlib/Analysis/SpecialFunctions/Log/Basic.lean,Mathlib/Analysis/SpecialFunctions/Log/Monotone.lean,Mathlib/Analysis/SpecialFunctions/Pow/Deriv.lean,Mathlib/Analysis/SpecialFunctions/Pow/Real.lean,Mathlib/Analysis/SpecificLimits/FloorPow.lean,Mathlib/MeasureTheory/Covering/BesicovitchVectorSpace.lean,Mathlib/MeasureTheory/Measure/Lebesgue/VolumeOfBalls.lean,Mathlib/NumberTheory/Modular.lean,Mathlib/NumberTheory/Transcendental/Liouville/LiouvilleWith.lean,Mathlib/Probability/Distributions/Pareto.lean |
30 |
29 |
['github-actions', 'grunweg', 'hrmacbeth', 'jcommelin', 'leanprover-bot', 'mathlib4-dependent-issues-bot'] |
nobody |
272-83740 8 months ago |
272-83740 8 months ago |
3-30853 3 days |
18748 |
FR-vdash-bot author:FR-vdash-bot |
refactor: deprecate `ContinuousLinearMapClass` |
---
- [ ] depends on: #18689
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-topology
merge-conflict
label:t-algebra$ |
115/49 |
Mathlib/Analysis/CStarAlgebra/Spectrum.lean,Mathlib/Analysis/LocallyConvex/WeakOperatorTopology.lean,Mathlib/Analysis/Normed/Algebra/Spectrum.lean,Mathlib/Analysis/Normed/Operator/LinearIsometry.lean,Mathlib/Topology/Algebra/Module/Basic.lean,Mathlib/Topology/Algebra/Module/CharacterSpace.lean,Mathlib/Topology/Algebra/Module/FiniteDimension.lean,Mathlib/Topology/Algebra/Module/StrongTopology.lean,Mathlib/Topology/Algebra/Module/WeakDual.lean,Mathlib/Topology/Homeomorph.lean |
10 |
5 |
['FR-vdash-bot', 'github-actions', 'leanprover-bot', 'mathlib4-dependent-issues-bot'] |
nobody |
270-74358 8 months ago |
270-74361 8 months ago |
0-989 16 minutes |
8686 |
j-loreaux author:j-loreaux |
refactor: allow non-unital `AlgEquiv` |
This refactors `AlgEquiv` (and `AlgEquivClass`) to incorporate a `map_smul` field instead of `commutes`. This allows us to weaken the type class assumptions on `AlgEquiv` from:
```lean
structure AlgEquiv (R A B : Type*) [CommSemiring R] [Semiring A] [Semiring B]
[Algebra R A] [Algebra R B]
```
to:
```lean
structure AlgEquiv (R A B : Type*) [Add A] [Add B] [Mul A] [Mul B] [SMul R A] [SMul R B]
```
in accordance with the other `Equiv` structures (e.g., `MulEquiv`, `AddEquiv`, `RingEquiv`). This allows us to use `AlgEquiv` for both unital and non-unital (even non-associative) algebra homomorphisms. Note in addition that `StarAlgEquiv` already follows this paradigm.
We supply the convenience constructor `AlgEquiv.ofCommutes`, which is marked `inline` and `reducible`, so that users can still provide go via the `commutes` route for constructing and `AlgEquiv` whenever it is more convenient.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
WIP
label:t-algebra$ |
286/227 |
Mathlib/Algebra/Algebra/Equiv.lean,Mathlib/Algebra/Algebra/Opposite.lean,Mathlib/Algebra/Algebra/Pi.lean,Mathlib/Algebra/Algebra/Subalgebra/Basic.lean,Mathlib/Algebra/Algebra/Tower.lean,Mathlib/Algebra/Category/AlgebraCat/Basic.lean,Mathlib/Algebra/DualQuaternion.lean,Mathlib/Algebra/MonoidAlgebra/Basic.lean,Mathlib/Algebra/MonoidAlgebra/ToDirectSum.lean,Mathlib/Algebra/Quaternion.lean,Mathlib/Algebra/Star/Free.lean,Mathlib/Algebra/Star/StarAlgHom.lean,Mathlib/Analysis/NormedSpace/LpEquiv.lean,Mathlib/Data/Complex/Module.lean,Mathlib/Data/IsROrC/Basic.lean,Mathlib/Data/Matrix/Basic.lean,Mathlib/Data/Matrix/DualNumber.lean,Mathlib/Data/MvPolynomial/Equiv.lean,Mathlib/Data/MvPolynomial/Rename.lean,Mathlib/Data/Polynomial/AlgebraMap.lean,Mathlib/LinearAlgebra/Matrix/Basis.lean,Mathlib/LinearAlgebra/Matrix/Charpoly/Coeff.lean,Mathlib/LinearAlgebra/Matrix/Reindex.lean,Mathlib/LinearAlgebra/Matrix/ToLin.lean,Mathlib/LinearAlgebra/TensorProduct/Opposite.lean,Mathlib/Logic/Equiv/TransferInstance.lean,Mathlib/RingTheory/FinitePresentation.lean,Mathlib/RingTheory/GradedAlgebra/Basic.lean,Mathlib/RingTheory/Ideal/QuotientOperations.lean,Mathlib/RingTheory/Localization/Basic.lean,Mathlib/RingTheory/MatrixAlgebra.lean,Mathlib/RingTheory/Polynomial/Quotient.lean,Mathlib/RingTheory/PolynomialAlgebra.lean,Mathlib/RingTheory/TensorProduct.lean,Mathlib/Topology/LocallyConstant/Algebra.lean |
35 |
2 |
['eric-wieser', 'j-loreaux'] |
nobody |
267-86153 8 months ago |
647-48930 1 year ago |
0-0 0 seconds |
11142 |
hmonroe author:hmonroe |
feat(ProofTheory): Define logical symbols abstractly; opens new top-level section, drawing from lean4-logic |
---
[](https://gitpod.io/from-referrer/)
|
t-logic
merge-conflict
awaiting-author
|
468/1 |
Mathlib.lean,Mathlib/Data/Fin/VecNotation.lean,Mathlib/ProofTheory/LogicSymbol.lean |
3 |
19 |
['PatrickMassot', 'YaelDillies', 'avigad', 'fpvandoorn', 'github-actions'] |
nobody |
267-7160 8 months ago |
267-7160 8 months ago |
92-18232 92 days |
11210 |
hmonroe author:hmonroe |
Test commit |
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict
WIP
|
1950/1 |
Mathlib.lean,Mathlib/Data/Fin/VecNotation.lean,Mathlib/ProofTheory/Calculus.lean,Mathlib/ProofTheory/FirstOrder/Arith/Language.lean,Mathlib/ProofTheory/FirstOrder/Basic/Syntax/Term.lean,Mathlib/ProofTheory/LogicSymbol.lean,Mathlib/ProofTheory/Matrix.lean,Mathlib/ProofTheory/Semantics.lean,Mathlib/ProofTheory/System.lean,docs/references.bib |
10 |
100 |
['github-actions'] |
nobody |
267-7159 8 months ago |
267-7159 8 months ago |
0-0 0 seconds |
18294 |
FR-vdash-bot author:FR-vdash-bot |
perf: make `Mul.toSMul` higher priority |
---
[](https://gitpod.io/from-referrer/)
|
awaiting-bench
t-algebra
merge-conflict
label:t-algebra$ |
2/5 |
Mathlib/Algebra/Group/Action/Defs.lean,Mathlib/Algebra/Order/Field/Pointwise.lean,Mathlib/Combinatorics/Additive/AP/Three/Defs.lean,Mathlib/Topology/Algebra/Module/WeakBilin.lean |
4 |
4 |
['FR-vdash-bot', 'github-actions', 'leanprover-bot'] |
nobody |
261-74752 8 months ago |
261-74753 8 months ago |
0-0 0 seconds |
19699 |
vihdzp author:vihdzp |
chore(SetTheory/Cardinal/Basic): tweak `#α = 0`, `#α = 1`, etc. lemmas |
We rename `le_one_iff_subsingleton` → `mk_le_one_iff` and `mk_le_one_iff_set_subsingleton` → `mk_set_le_one_iff` to match the names of other lemmas in this section. We also add `mk_eq_one_iff` and `mk_set_eq_one_iff`.
---
These last two lemmas can probably be golfed somehow.
[](https://gitpod.io/from-referrer/)
|
t-set-theory
awaiting-CI
merge-conflict
|
48/16 |
Mathlib/SetTheory/Cardinal/Basic.lean |
1 |
1 |
['github-actions'] |
nobody |
259-80186 8 months ago |
259-80186 8 months ago |
0-5976 1 hour |
15773 |
kkytola author:kkytola |
feat: Add type class for ENat-valued floor functions |
This PR adds a type class for extended natural number -valued floor functions. This is split off from #15269, where the suggestions were to make the floor function on ENNReal ENat-valued and to have an API mimicling FloorSemirings. Besides ENNReal, at least ENNRat would naturally satisfy the general type class.
---
Two things are worth noting:
* To fully mimic `FloorSemiring` API, also ceiling functions need to be added. The plan is to do that in a later PR.
* The PR introduces the class `CastNatENatClass` to ensure that `natCast` and a coercion from `ENat` behave in the natural and order-respecing manner. This feels a little ad hoc, but such assumptions are needed for general `ENat`-valued floor functions to behave well.
[](https://gitpod.io/from-referrer/)
|
t-order
merge-conflict
awaiting-author
|
231/0 |
Mathlib.lean,Mathlib/Algebra/Order/EFloor.lean,Mathlib/Data/ENat/Basic.lean |
3 |
5 |
['YaelDillies', 'github-actions', 'kkytola', 'urkud'] |
nobody |
253-47926 8 months ago |
253-47926 8 months ago |
66-24436 66 days |
3251 |
kmill author:kmill |
feat: deriving `LinearOrder` for simple enough inductive types |
Uses the same machinery underlying the `Fintype` derive handler to derive a lexicographical `LinearOrder` for non-recursive inductive types that have no indices.
In principle more complicated types can have `LinearOrder`s, but that would require a more sophisticated implementation.
---
- [x] depends on: #3198
[](https://gitpod.io/from-referrer/)
|
t-meta
merge-conflict
awaiting-author
WIP
|
82/0 |
Mathlib.lean,Mathlib/Tactic/DeriveLinearOrder.lean |
2 |
5 |
['ChrisHughes24', 'kim-em', 'kmill', 'vihdzp'] |
nobody |
251-22579 8 months ago |
251-22579 8 months ago |
1-80342 1 day |
3610 |
TimothyGu author:TimothyGu |
feat: derive Infinite automatically for inductive types |
Deals with recursive types, but not mutually recursive types or types with indices right now. See docstring for details.
---
[](https://gitpod.io/from-referrer/)
|
t-meta
merge-conflict
awaiting-author
|
517/0 |
Mathlib.lean,Mathlib/Tactic/DeriveInfinite.lean,test/DeriveInfinite.lean |
3 |
11 |
['TimothyGu', 'digama0', 'eric-wieser', 'grunweg', 'kim-em', 'kmill'] |
kmill assignee:kmill |
251-22578 8 months ago |
251-22578 8 months ago |
8-36622 8 days |
16120 |
awainverse author:awainverse |
feat(ModelTheory/Algebra/Ring/Basic): Ring homomorphisms are a `StrongHomClass` for the language of rings |
Adds an `IsAlgebraic` instance to the language of rings
Adds a `StrongHomClass` instance to the type of ring homomorphisms between rings with `CompatibleRing` structures
---
[](https://gitpod.io/from-referrer/)
|
t-logic
t-algebra
RFC
merge-conflict
label:t-algebra$ |
34/13 |
Mathlib/ModelTheory/Algebra/Ring/Basic.lean |
1 |
10 |
['ChrisHughes24', 'YaelDillies', 'awainverse', 'github-actions', 'jcommelin'] |
nobody |
249-40119 8 months ago |
249-40119 8 months ago |
135-29017 135 days |
15045 |
Command-Master author:Command-Master |
fix(LinearAlgebra/Alternating/Basic): fix `MultilinearMap.alternatization` |
See https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/kernel.20deep.20recursion.20detected.
Fix
```lean
import Mathlib.LinearAlgebra.Determinant
example : (1 : Matrix (Fin 8) (Fin 8) ℚ).det = 1 := by
rw [Matrix.det_one]
```
causing a `(kernel) deep recursion detected` error.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
awaiting-author
label:t-algebra$ |
51/21 |
Mathlib/Data/Nat/Factorial/SuperFactorial.lean,Mathlib/LinearAlgebra/Alternating/Basic.lean,test/DetOne.lean |
3 |
12 |
['Command-Master', 'PatrickMassot', 'eric-wieser', 'github-actions', 'grhkm21', 'grunweg', 'kbuzzard', 'kim-em'] |
nobody |
249-7408 8 months ago |
249-7409 8 months ago |
0-8789 2 hours |
20527 |
trivial1711 author:trivial1711 |
refactor(Topology/UniformSpace/Completion): more descriptive names for `α → Completion α` |
- We rename the various maps `α → Completion α` in order to make their names more consistent.
- Let `α` be a uniform space. We rename the uniformly continuous function `α → Completion α` from `UniformSpace.Completion.coe'` to `UniformSpace.Completion.coe`.
- Let `α` be a uniform additive group. We rename the additive group homomorphism `α →+ Completion α` from `UniformSpace.Completion.toCompl` to `UniformSpace.Completion.coeAddHom`.
- Let `α` be a uniform ring. The ring homomorphism `α →+* Completion α` is called `UniformSpace.Completion.coeRingHom`; its name is unchanged.
- Let `α` be a normed space over a field `𝕜`. We rename the linear isometry `α →ₗᵢ[𝕜] Completion α` from `UniformSpace.Completion.toComplₗᵢ` to `UniformSpace.Completion.coeₗᵢ`.
- Let `α` be a normed space over a field `𝕜`. We rename the continuous linear map `α →L[𝕜] Completion α` from `UniformSpace.Completion.toComplL` to `UniformSpace.Completion.coeL`.
- Let `α` be a normed additive group. We rename the norm preserving homomorphism `NormedAddGroupHom α (Completion α)` from `NormedAddCommGroup.toCompl` to `UniformSpace.Completion.coeNormedAddGroupHom`.
- We analogously rename some other theorems.
- We add some trivial theorems (all of which are proved by `rfl`) that state that the functions considered above are equal. We give all of them the `simp` and `norm_cast` attributes.
- We add a new theorem `UniformSpace.Completion.coeAddHom_eq_coe` that states that `UniformSpace.Completion.coeAddHom` and `UniformSpace.Completion.coe` are equal as functions.
- We similarly add a new theorem `UniformSpace.Completion.coeRingHom_eq_coe`.
- We rename the theorem `UniformSpace.Completion.coe_toComplₗᵢ` to `UniformSpace.Completion.coeₗᵢ_eq_coe`.
- We rename the theorem `UniformSpace.Completion.coe_toComplL` to `UniformSpace.Completion.coeL_eq_coe`.
- We similarly add a new theorem `UniformSpace.Completion.coeNormedAddGroupHom_eq_coe`.
- We change all occurrences of the string `((↑) : α → Completion α)` to `(coe : α → Completion α)` or just `coe`.
- We put the statements of some theorems into simp normal form by using the plain function `coe` rather than the homomorphisms that carry more structure.
---
[](https://gitpod.io/from-referrer/)
|
t-topology
merge-conflict
|
130/92 |
Mathlib/Analysis/Analytic/Uniqueness.lean,Mathlib/Analysis/Calculus/FDeriv/Analytic.lean,Mathlib/Analysis/Complex/AbsMax.lean,Mathlib/Analysis/Complex/Liouville.lean,Mathlib/Analysis/InnerProductSpace/Completion.lean,Mathlib/Analysis/Normed/Group/HomCompletion.lean,Mathlib/Analysis/Normed/Module/Completion.lean,Mathlib/Analysis/SpecialFunctions/NonIntegrable.lean,Mathlib/MeasureTheory/Integral/IntegralEqImproper.lean,Mathlib/Topology/Algebra/GroupCompletion.lean,Mathlib/Topology/Algebra/InfiniteSum/GroupCompletion.lean,Mathlib/Topology/Algebra/InfiniteSum/Nonarchimedean.lean,Mathlib/Topology/Algebra/Nonarchimedean/Completion.lean,Mathlib/Topology/Algebra/UniformRing.lean,Mathlib/Topology/Category/UniformSpace.lean,Mathlib/Topology/MetricSpace/Completion.lean,Mathlib/Topology/UniformSpace/Completion.lean |
17 |
4 |
['eric-wieser', 'github-actions', 'trivial1711'] |
nobody |
242-71151 7 months ago |
242-71151 7 months ago |
6-66637 6 days |
17739 |
Aaron1011 author:Aaron1011 |
feat(Topology/Order/DenselyOrdered): prove Not (IsOpen) for intervals |
Prove that Iic/Ici/Ioc/Ico/Icc intervals are not open in densely ordered topologies with no min/max element
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-topology
merge-conflict
awaiting-author
|
27/0 |
Mathlib/Topology/Order/DenselyOrdered.lean |
1 |
8 |
['github-actions', 'vihdzp'] |
nobody |
240-58426 7 months ago |
240-58426 7 months ago |
0-4704 1 hour |
18474 |
FR-vdash-bot author:FR-vdash-bot |
perf: lower the priority of `*WithOne.to*` instances |
---
From #7873.
[](https://gitpod.io/from-referrer/)
|
t-data
slow-typeclass-synthesis
t-algebra
merge-conflict
label:t-algebra$ |
9/2 |
Mathlib/Algebra/Polynomial/BigOperators.lean,Mathlib/Data/Int/Cast/Defs.lean,Mathlib/Data/Nat/Cast/Defs.lean |
3 |
7 |
['FR-vdash-bot', 'eric-wieser', 'github-actions', 'leanprover-bot'] |
nobody |
240-58181 7 months ago |
240-58181 7 months ago |
76-67978 76 days |
20656 |
Komyyy author:Komyyy |
feat(Mathlib/Geometry/Manifold/VectorBundle/Sphere): convert orthogonal smooth `M → 𝕊ⁿ` & `M → ℝⁿ⁺¹` to smooth `M → T𝕊ⁿ` |
Current Mathlib has no easy way to define function from a manifold to tangent bundles of sphere: `T𝕊ⁿ`.
This PR gives this: `sphereTangentMap`. This convert orthogonal smooth `M → 𝕊ⁿ` & `M → ℝⁿ⁺¹` to smooth `M → T𝕊ⁿ`.
I also proved that if `f : M → 𝕊ⁿ` & `g : M → ℝⁿ⁺¹` are smooth then `sphereTangentMap` of `f` & `g` is smooth too.
---
⚠ **CAUTION**
I formalized this in my spare time.
I don't have the energy to maintain the PR, but I create this PR so this may helps everyone.
The only one thing to do is proof cleanup.
TODO:
- [x] `contDiff_uncurry_stereoInvFunAux` & `coe_sphere_comp_stereoInvFun` may have to be moved to `Mathlib.Geometry.Manifold.Instances.Sphere`.
- [ ] Proof cleanup. Current proof may be redundant and ugly.
[](https://gitpod.io/from-referrer/)
|
t-differential-geometry
merge-conflict
please-adopt
|
246/6 |
Mathlib.lean,Mathlib/Geometry/Manifold/Instances/Sphere.lean,Mathlib/Geometry/Manifold/VectorBundle/Sphere.lean |
3 |
1 |
['github-actions'] |
nobody |
240-6715 7 months ago |
240-6715 7 months ago |
0-0 0 seconds |
15711 |
znssong author:znssong |
feat(Combinatorics/SimpleGraph): Some lemmas about walk, cycle and Hamiltonian cycle |
---
These lemmas are separated from the `meow-sister/BondyChvatal` branch and will be needed for the proof of the Bondy-Chvátal theorem.
- [x] depends on: #15536
- [x] depends on: #16294 |
new-contributor
t-combinatorics
merge-conflict
awaiting-author
|
407/3 |
Mathlib/Combinatorics/SimpleGraph/Finite.lean,Mathlib/Combinatorics/SimpleGraph/Hamiltonian.lean,Mathlib/Combinatorics/SimpleGraph/Path.lean,Mathlib/Combinatorics/SimpleGraph/Walk.lean |
4 |
22 |
['Rida-Hamadani', 'YaelDillies', 'github-actions', 'mathlib4-dependent-issues-bot', 'znssong'] |
nobody |
239-77512 7 months ago |
239-77512 7 months ago |
9-13962 9 days |
18629 |
tomaz1502 author:tomaz1502 |
feat(Computability.Timed): Formalization of runtime complexity of List.merge |
This PR adds the formalization of the runtime complexity of the merge function, defined in `Data/List/Sort`.
Requires: https://github.com/leanprover-community/mathlib4/pull/15450
References:
- Previous PR on mathlib3: https://github.com/leanprover-community/mathlib3/pull/14494/
- First discussion on Zulip: https://leanprover.zulipchat.com/#narrow/stream/113488-general/topic/BSc.20Final.20Project/near/220647062
- Second disussion on Zulip: https://leanprover.zulipchat.com/#narrow/stream/113488-general/topic/Formalization.20of.20Runtime.20Complexity.20of.20Sorting.20Algorithms/near/284184450
---
[](https://gitpod.io/from-referrer/)
|
t-computability
new-contributor
merge-conflict
awaiting-author
|
186/0 |
Mathlib.lean,Mathlib/Computability/Timed/InsertionSort.lean,Mathlib/Computability/Timed/Merge.lean |
3 |
2 |
['github-actions', 'trivial1711'] |
nobody |
239-43431 7 months ago |
239-43431 7 months ago |
33-11262 33 days |
8362 |
urkud author:urkud |
feat(Asymptotics): define `ReflectsGrowth` |
---
- [x] depends on: #8349
[](https://gitpod.io/from-referrer/)
|
t-analysis
merge-conflict
awaiting-author
|
268/0 |
Mathlib.lean,Mathlib/Analysis/Asymptotics/ReflectsGrowth.lean |
2 |
14 |
['YaelDillies', 'fpvandoorn', 'github-actions', 'leanprover-community-mathlib4-bot', 'urkud'] |
nobody |
237-50685 7 months ago |
237-50685 7 months ago |
1-41158 1 day |
6692 |
prakol16 author:prakol16 |
feat: disjoint indexed union of local homeomorphisms |
Add disjoint indexed union of local equivs and local homeomorphisms
---
This is leading up to PRing some things related to covering spaces that I wrote a long time ago in lean 3 but never submitted a PR for. Note that this was converted using mathport.
[](https://gitpod.io/from-referrer/)
|
t-topology
merge-conflict
awaiting-author
|
126/0 |
Mathlib/Logic/Equiv/PartialEquiv.lean,Mathlib/Topology/PartialHomeomorph.lean |
2 |
4 |
['alreadydone', 'github-actions', 'winstonyin'] |
nobody |
237-35281 7 months ago |
237-35281 7 months ago |
117-22351 117 days |
19291 |
PieterCuijpers author:PieterCuijpers |
feat(Algebra/Order/Hom): add quantale homomorphism |
Definition of quantale homomorphisms as functions that are both semigroup homomorphisms and complete lattice homomorphisms.
---
- [x] depends on: #19810
- [x] depends on: #19811
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-algebra
merge-conflict
awaiting-author
label:t-algebra$ |
209/0 |
Mathlib.lean,Mathlib/Algebra/Order/Hom/Quantale.lean,scripts/noshake.json |
3 |
29 |
['PieterCuijpers', 'YaelDillies', 'github-actions', 'kim-em', 'mathlib4-dependent-issues-bot'] |
nobody |
234-65090 7 months ago |
234-65091 7 months ago |
36-2255 36 days |
19352 |
hrmacbeth author:hrmacbeth |
chore: change some `nlinarith`s to `linear_combination`s |
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict
WIP
|
13/13 |
Archive/Imo/Imo2021Q1.lean,Archive/Wiedijk100Theorems/AreaOfACircle.lean,Mathlib/Analysis/Normed/Group/AddCircle.lean,Mathlib/Analysis/Normed/Group/Basic.lean,Mathlib/Analysis/Normed/Ring/Units.lean,Mathlib/Analysis/SpecialFunctions/Complex/LogBounds.lean,Mathlib/Combinatorics/SimpleGraph/Regularity/Increment.lean,Mathlib/NumberTheory/Modular.lean |
8 |
4 |
['github-actions', 'hrmacbeth', 'leanprover-bot'] |
nobody |
233-7901 7 months ago |
233-7901 7 months ago |
0-8636 2 hours |
20372 |
jvlmdr author:jvlmdr |
feat(MeasureTheory/Function): Add ContinuousLinearMap.bilinearCompLp(L) |
Introduce ContinuousLinearMap.bilinearCompLp and bilinearCompLpL.
Generalize eLpNorm_le_eLpNorm_mul_eLpNorm theorems to include constant C in bound condition.
---
Expect this may be useful for defining tempered distributions from functions in `L^p`.
The definitions more or less follow `ContinuousLinearMap.compLp...`. Names are loosely analogous to `ContinuousLinearMap.bilinearComp` and `SchwartzMap.bilinLeftCLM`.
Note: I preferred the spelling `hpqr : p⁻¹ + q⁻¹ = r⁻¹` with `f` in `L^p` and `g` in `L^q` to `hpqr : 1 / p = 1 / q + 1 / r`. It's easier to obtain from `ENNReal.IsConjExponent` too.
A few questions:
- [ ] I defined `bilinear{Left,Right}LpL` in addition to `bilinearCompLpL` because `LinearMap.mkContinuous₂` is marked as `noncomputable` and `LinearMap.mkContinuous` is not. Is this worth the extra definitions? (Note: This is not visible in the source due to `noncomputable section`.)
- [ ] Should I use `C : ℝ` instead of `C : NNReal` for `eLpNorm_le_eLpNorm_mul_eLpNorm'_of_norm'`?
- [ ] Is it going to be painful to have `[Fact (1 ≤ p)] [Fact (1 ≤ q)] [Fact (1 ≤ r)]`? I don't think there's a way to avoid it though. Maybe providing specialized versions for `p.IsConjExponent q` with `L^1`?
Naming:
- [ ] Is it satisfactory to add a `'` to the `eLpNorm_le_eLpNorm_mul_eLpNorm ` definitions in `CompareExp.lean` where `≤ ‖f x‖ * ‖g x‖` has been replaced with `≤ C * ‖f x‖ * ‖g x‖`? These could replace the existing theorems, although I don't want to break backwards compatibility. There are 5 instances: `eLpNorm_le_eLpNorm_top_mul_eLpNorm'`, `eLpNorm_le_eLpNorm_mul_eLpNorm_top'`, `eLpNorm'_le_eLpNorm'_mul_eLpNorm''`, `eLpNorm_le_eLpNorm_mul_eLpNorm_of_nnnorm'`, `eLpNorm_le_eLpNorm_mul_eLpNorm'_of_norm'` (I'm not sure why the existing theorem `eLpNorm_le_eLpNorm_mul_eLpNorm'_of_norm` has an internal `'`)
- [ ] Is `bilinearLeftLpL` a suitable name? Other options: `bilinearCompLpLeftL`, `bilinearCompLeftLpL`, `bilinLeftLpL` (analogous to `SchwartzMap.bilinLeftCLM`)
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-measure-probability
merge-conflict
|
203/40 |
Mathlib/MeasureTheory/Function/LpSeminorm/CompareExp.lean,Mathlib/MeasureTheory/Function/LpSpace.lean |
2 |
1 |
['github-actions'] |
nobody |
227-82438 7 months ago |
227-82438 7 months ago |
27-43617 27 days |
17176 |
arulandu author:arulandu |
feat: integrals and integrability with .re |
Lemmas for swapping order of .re and integration/integrability.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-measure-probability
merge-conflict
awaiting-author
|
49/0 |
Mathlib/MeasureTheory/Function/L1Space.lean,Mathlib/MeasureTheory/Integral/IntegrableOn.lean,Mathlib/MeasureTheory/Integral/IntervalIntegral.lean,Mathlib/MeasureTheory/Integral/SetIntegral.lean |
4 |
30 |
['EtienneC30', 'arulandu', 'github-actions', 'loefflerd'] |
nobody |
226-56871 7 months ago |
226-56871 7 months ago |
9-73631 9 days |
20872 |
grunweg author:grunweg |
feat: lint against the tactic.skipAssignedInstances option in mathlib |
This means we can remove the corresponding technical debt entry. We also correct some outdated details in the Linter/Style.lean docstring.
---
[](https://gitpod.io/from-referrer/)
|
tech debt
t-linter
merge-conflict
awaiting-author
|
63/7 |
Mathlib/Analysis/InnerProductSpace/PiL2.lean,Mathlib/Tactic/Linter/Style.lean,Mathlib/Topology/Separation/Regular.lean,MathlibTest/LintStyle.lean,scripts/technical-debt-metrics.sh |
5 |
17 |
['adomani', 'github-actions', 'grunweg'] |
nobody |
226-50901 7 months ago |
226-50901 7 months ago |
0-9411 2 hours |
2605 |
eric-wieser author:eric-wieser |
chore: better error message in linarith |
On this mwe:
```lean
import Mathlib.Tactic.Linarith
example (s : Set ℕ) (h : s = s) : 0 ≤ 1 :=
by linarith
```
this now indicates where the internal error is coming from.
Is there a better way of chaining errors than this?
---
[](https://gitpod.io/from-referrer/)
|
t-meta
merge-conflict
awaiting-author
|
12/1 |
Mathlib/Tactic/Linarith/Preprocessing.lean |
1 |
3 |
['Vierkantor', 'harahu', 'kim-em', 'mo271'] |
nobody |
225-73031 7 months ago |
660-46318 1 year ago |
4-7271 4 days |
11837 |
trivial1711 author:trivial1711 |
feat: completion of a uniform multiplicative group |
Multiplicativize `Topology.Algebra.GroupCompletion`. That is, rewrite it in the multiplicative setting and recover the original results using `@[to_additive]`.
- Because `@[to_additive]` doesn't work with `noncomputable section` (https://github.com/leanprover/lean4/pull/2610), some instances with `@[to_additive]` need to be explicitly marked with `noncomputable instance`.
- One might be tempted to multiplicativize this definition from `Topology.Algebra.GroupCompletion`:
```lean
instance [UniformSpace α] [Add α] : Add (Completion α) :=
⟨Completion.map₂ (· + ·)⟩
```
to this:
```lean
@[to_additive]
instance [UniformSpace α] [Mul α] : Mul (Completion α) :=
⟨Completion.map₂ (· * ·)⟩
```
However, as Eric Wieser pointed out, doing so would create a bad diamond with the definition
```lean
instance [UniformSpace α] [TopologicalRing α] [UniformAddGroup α] [Ring α] : Mul (Completion α) :=
⟨curry <| (denseInducing_coe.prod denseInducing_coe).extend ((↑) ∘ uncurry (· * ·))⟩
```
in `Topology.Algebra.UniformRing`.
How should this diamond be resolved? Well, the definition of multiplication that uses `curry <| (denseInducing_coe.prod denseInducing_coe).extend ((↑) ∘ uncurry (· * ·))` is the "correct" one. For example, it yields the correct result if `α` is `ℚ`, unlike the definition that uses `Completion.map₂ (· * ·)`. (This is because `Completion.map₂` yields junk values if used on a function which is not uniformly continuous. Note, however, that if multiplication on `α` *is* uniformly continuous, then `Completion.map₂ (· * ·)` and `curry <| (denseInducing_coe.prod denseInducing_coe).extend ((↑) ∘ uncurry (· * ·))` are propositionally equal.) So, following Eric's suggestion, we remove the definition that uses `Completion.map₂ (· * ·)`, and generalize the other definition to any uniform space with a multiplication operation:
```lean
@[to_additive]
noncomputable instance [UniformSpace α] [Mul α] : Mul (Completion α) :=
⟨curry <| (denseInducing_coe.prod denseInducing_coe).extend ((↑) ∘ uncurry (· * ·))⟩
```
This requires slightly modifying some of the proofs in `Topology.Algebra.GroupCompletion`. For example, suppose that `α` is a uniform group. Since we can no longer use `Completion.continuous_map₂`, it becomes more efficient to prove that the multiplication, inversion, and division operations on `Completion α` are uniformly continuous *before* we prove that `Completion α` is a group.
- Previously, `Topology.Algebra.GroupCompletion` had an instance:
```lean
instance [UniformSpace α] [Sub α] : Sub (Completion α) := ...
```
Naively multiplicativizing this would yield
```lean
@[to_additive]
instance [UniformSpace α] [Inv α] : Inv (Completion α) := ...
```
Unfortunately, this would conflict with `Topology.Algebra.UniformField`, which already instantiates `Inv (Completion α)` when `α` is a uniform field. Instead, we use two different `instance` declarations. (If `α` is an additive group, then this instantiates `Neg (Completion α)` twice, and the instances are syntactically equal.)
```lean
@[to_additive]
noncomputable instance [UniformSpace α] [Group α] : Inv (Completion α) := ...
instance [UniformSpace α] [Neg α] : Neg (Completion α) := ...
```
This avoids the bad diamond (because a uniform field can never be a `Group`) while remaining backward compatible. Note that the `@[to_additive]` is necessary here, because it maintains the link between the additive setting and multiplicative setting. We use a similar method to instantiate `Div (Completion α)`.
- Some definitions in this file involve a module structure on `α`. We leave these as is and do not attempt to multiplicativize them at all.
- The instance of `DistribMulAction` must be multiplicativized to an instance of `MulDistribMulAction` manually.
Zulip thread: https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/Completion.20of.20a.20uniform.20multiplicative.20group
---
# (Small) Issue
Recall the following trick that this pull request uses to define inversion and negation on uniform spaces. The idea is that we define negation on the completion of any uniform space that has a negation operation, but we define inversion on only the completion of a uniform space that has the structure of a multiplicative group. We do this to avoid creating a bad diamond with the inversion operation on a uniform field.
```lean
@[to_additive]
noncomputable instance {α : Type*} [UniformSpace α] [Group α] : Inv (Completion α) := ...
instance {α : Type*} [UniformSpace α] [Neg α] : Neg (Completion α) := ...
```
Now, suppose that we want to prove `coe_inv_of_group` (resp. `coe_neg`), which states that the coercion `α → Completion α` commutes with inversion (resp. negation). In the current version of this pull request, `coe_inv_of_group` (resp. `coe_neg`) only applies to uniform multiplicative (resp. additive) groups. However, we do not use the fact that multiplication (resp. addition) on `α` is uniformly continuous to prove it. We only use the fact that inversion (resp. negation) is continuous. So, what we really want is to have more general statements that look like this:
```lean
theorem coe_inv_of_group {α : Type*} [UniformSpace α] [Group α] [ContinuousInv α] : ...
theorem coe_neg {α : Type*} [UniformSpace α] [Neg α] [ContinuousNeg α] : ...
```
Note that `coe_inv_of_group` needs the assumption `[Group α]`, because otherwise inversion is not defined on `Completion α` at all. However, `coe_neg` does not need the analogous assumption `[AdditiveGroup α]`.
The question is: If `coe_inv_of_group` and `coe_neg` are written in this more general form, how can we link them using `@[to_additive]`? Here is one option, but it obviously leaves something to be desired.
```lean
@[to_additive coe_neg_do_not_use_this_use_the_more_general_version]
theorem coe_inv_of_group {α : Type*} [UniformSpace α] [Group α] [ContinuousInv α] : ...
theorem coe_neg {α : Type*} [UniformSpace α] [Neg α] [ContinuousNeg α] : ...
```
Co-authored-by: Eric Wieser
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-topology
merge-conflict
WIP
help-wanted
label:t-algebra$ |
342/217 |
Mathlib/Analysis/InnerProductSpace/Completion.lean,Mathlib/Analysis/Normed/Group/HomCompletion.lean,Mathlib/Analysis/Normed/Module/Completion.lean,Mathlib/Topology/Algebra/GroupCompletion.lean,Mathlib/Topology/Algebra/InfiniteSum/GroupCompletion.lean,Mathlib/Topology/Algebra/Nonarchimedean/Completion.lean,Mathlib/Topology/Algebra/UniformField.lean,Mathlib/Topology/Algebra/UniformMulAction.lean,Mathlib/Topology/Algebra/UniformRing.lean |
9 |
14 |
['eric-wieser', 'github-actions', 'trivial1711'] |
nobody |
225-50536 7 months ago |
225-50536 7 months ago |
101-64856 101 days |
14799 |
luigi-massacci author:luigi-massacci |
feat(Analysis/MeanInequalities): Weighted QM-AM inequality |
The inequality between the quadratic and arithmetic mean as a consequence of Jensen's inequality. Weighted version for positive real valued functions from a `Finset`. Fix notation for sums, switching to `∈` in place of `in`.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-analysis
easy
merge-conflict
awaiting-author
|
26/3 |
Mathlib/Analysis/MeanInequalities.lean |
1 |
8 |
['YaelDillies', 'acmepjz', 'github-actions', 'luigi-massacci', 'vihdzp'] |
nobody |
225-50042 7 months ago |
225-50042 7 months ago |
0-38862 10 hours |
14686 |
smorel394 author:smorel394 |
feat (AlgebraicGeometry/Grassmannian): define the Grassmannian scheme |
# The Grassmannian scheme
Define the Grassmannian scheme by gluing affine charts.
We fix a commutative ring `K`, a free `K`-module of finite type `V` and two natural numbers
`r` and `c`. The scheme we define should parametrize surjective `K`-linear maps
`V →ₗ[K] (Fin r → K)`, assuming that `V` is of rank `r + c`. We actually define the scheme
without assuming the condition on the rank of `V`, but it is empty unless the rank of `V` is
`r + c`.
Main definitions:
* `Grassmannian.glueData K V r c`: the `AlgebraicGeometry.Scheme.GlueData` defining the
Grassmannian scheme.
* `Grassmannian K V r c`: the Grassmannian scheme, defined as
`(Grassmannian.glueData K V r c).glued`.
* `Grassmannian.structMorphism K V r c`: the structural morphism from `Grassmannian K V r c`
to `Spec K`.
# Implementation
We use as index type for the charts the type `Basis (Fin (r + c)) K V` (so this is empty unless
`V` is free of rank `r + c`). All the charts are the same and equal to the affine space with
coordinates indexed by `Fin c × Fin r`, that is, to `Spec (MvPolynomial (Fin c × Fin r) K)`.
The idea is that, for `i` in `Basis (Fin (r + c)) K V`, the corresponding chart will
parametrize all surjective `K`-linear maps `φ : V →ₗ[K] (Fin r → K)` that become isomorphisms
when restricted to the `K`-submodule generated by the first `r` vectors of the basis `i`.
To get the point of the chart corresponding to `φ`, we take the matrix of `φ` in the basis `i` of
`V` and the canonical basis of `Fin r → K`, we divide it on the right by its top `r × r`
square submatrix (which is invertible by assumption), and we taken the botton `c × r`
submatrix.
This is almost the usual description of the Grassmannian by charts, with three differences:
* We consider the Grassmannian parametrizing `r`-dimensional quotients of `V` instead of
`r`-dimensional subspaces of `V`, because this is more natural when working over a general
ring (or scheme).
* In the usual description, we fix a basis of `V` and index the chart by its subsets `I` of
cardinality `r`. Here, to avoid making a choice, we instead index charts by the set of
bases of `V` and always choose the subset `I` to consist of the first `r` vectors.
* Instead of working with `FiniteDimensional.finrank K V - r`, which would cause technical
trouble because of the way subtraction works on `ℕ`, we introduce the codimension `c` as an
auxiliary variable, and our constructions are only interesting when `r + c` is equal to
`FiniteDimensional.finrank K V`.
# Why is this a WIP
* There a bunch of lemmas in the file `AlgebraicGeometry/Grassmannian/Lemmas.lean` that either should not be necessary or should be put in another PR for some other part of mathlib.
* The proofs in `AlgebraicGeometry/Grassmannian/Basic.lean` are probably too complicated, and the names suck.
# Notes.
This contribution was created as part of the AIM workshop "Formalizing algebraic geometry" in
June 2024.
---
- [x] depends on: #14711
[](https://gitpod.io/from-referrer/)
|
workshop-AIM-AG-2024
t-algebraic-geometry
merge-conflict
please-adopt
WIP
|
1002/0 |
Mathlib.lean,Mathlib/AlgebraicGeometry/Grassmannian/Basic.lean,Mathlib/AlgebraicGeometry/Grassmannian/Lemmas.lean |
3 |
15 |
['erdOne', 'github-actions', 'joelriou', 'leanprover-community-mathlib4-bot', 'smorel394'] |
nobody |
221-10962 7 months ago |
221-10962 7 months ago |
0-201 3 minutes |
9449 |
hmonroe author:hmonroe |
feat: Add Turing machine with the quintet definition (TMQ) and a chainable step function for each TM type |
---
[](https://gitpod.io/from-referrer/)
|
t-computability
merge-conflict
awaiting-author
|
458/1 |
Mathlib/Computability/TuringMachine.lean,Mathlib/Logic/PartArith.lean |
2 |
8 |
['eric-wieser', 'github-actions', 'hmonroe'] |
nobody |
220-15215 7 months ago |
220-15215 7 months ago |
14-19968 14 days |
18719 |
FR-vdash-bot author:FR-vdash-bot |
perf: lower the priority of `SemilinearMapClass.toAddHomClass` |
---
[](https://gitpod.io/from-referrer/)
|
awaiting-bench
slow-typeclass-synthesis
t-algebra
merge-conflict
label:t-algebra$ |
14/7 |
Mathlib/Algebra/Module/LinearMap/Defs.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Unique.lean,MathlibTest/TCSynth.lean |
3 |
4 |
['FR-vdash-bot', 'github-actions', 'leanprover-bot'] |
nobody |
218-76432 7 months ago |
218-76432 7 months ago |
0-0 0 seconds |
20663 |
EtienneC30 author:EtienneC30 |
feat: `PFunLike` typeclass for partial homomorphisms and `LinearPMapClass` |
A test PR implementing a typeclass `PFunLike` to represent partial homomorphisms and building a `LinearPMapClass` typeclass. Started from [this](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/ContinuousLinearPMap) discussion.
---
[](https://gitpod.io/from-referrer/)
|
t-data
t-algebra
merge-conflict
WIP
label:t-algebra$ |
278/49 |
Mathlib.lean,Mathlib/Algebra/Group/PHom.lean,Mathlib/Algebra/Module/Injective.lean,Mathlib/Analysis/Convex/Cone/Extension.lean,Mathlib/Data/PFunLike.lean,Mathlib/GroupTheory/GroupAction/PHom.lean,Mathlib/LinearAlgebra/LinearPMap.lean |
7 |
1 |
['github-actions'] |
nobody |
217-68880 7 months ago |
217-68880 7 months ago |
0-0 0 seconds |
19697 |
quangvdao author:quangvdao |
feat(BigOperators/Fin): Sum/product over `Fin` intervals |
This PR adds new theorems about the sum/product of some vector over `Fin` intervals. One example is:
```
@[to_additive]
theorem prod_Iic_succ (i : Fin n) :
∏ j ∈ Iic i.succ, v j = (∏ j ∈ Iic i.castSucc, v j) * v i.succ
```
---
- [x] depends on: #20360
This is in preparation for reworking `finSigmaFinEquiv` and `finProdFinEquiv` in #19013.
[](https://gitpod.io/from-referrer/)
|
t-data
merge-conflict
awaiting-author
|
87/12 |
Mathlib/Algebra/BigOperators/Fin.lean,Mathlib/Data/Fintype/Fin.lean,Mathlib/Order/Interval/Finset/Fin.lean |
3 |
20 |
['Ruben-VandeVelde', 'YaelDillies', 'eric-wieser', 'github-actions', 'mathlib4-dependent-issues-bot', 'quangvdao'] |
nobody |
217-57633 7 months ago |
217-57633 7 months ago |
6-25961 6 days |
19353 |
hrmacbeth author:hrmacbeth |
chore: golf some term/rw proofs using `linear_combination` |
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict
WIP
|
47/102 |
Archive/Wiedijk100Theorems/SumOfPrimeReciprocalsDiverges.lean,Mathlib/Analysis/Convex/Slope.lean,Mathlib/Analysis/Seminorm.lean,Mathlib/MeasureTheory/Integral/RieszMarkovKakutani.lean,Mathlib/NumberTheory/Modular.lean,Mathlib/NumberTheory/Zsqrtd/Basic.lean,Mathlib/Topology/ContinuousMap/ZeroAtInfty.lean |
7 |
5 |
['github-actions', 'grunweg', 'hrmacbeth', 'leanprover-bot'] |
grunweg assignee:grunweg |
216-56754 7 months ago |
216-56754 7 months ago |
0-7781 2 hours |
21196 |
vihdzp author:vihdzp |
chore: make argument of `zero_le` implicit |
This simplifies our expressions probably 95% of the time, and the remaining 5% we can simply use the Lean 4 implicit argument notation.
---
[](https://gitpod.io/from-referrer/)
|
t-order
awaiting-CI
merge-conflict
|
10/10 |
Mathlib/Algebra/Order/Monoid/Canonical/Defs.lean |
1 |
1 |
['github-actions'] |
nobody |
216-32876 7 months ago |
216-32876 7 months ago |
0-0 0 seconds |
21610 |
JLimperg author:JLimperg |
Aesop forward benchmark: forward precomp |
Not a real PR, just for benchmarking.
|
merge-conflict |
30/27 |
Mathlib/Data/List/InsertIdx.lean,Mathlib/Tactic/Recall.lean,Mathlib/Topology/List.lean,Test.lean,lake-manifest.json,lakefile.lean,lean-toolchain |
7 |
3 |
['JLimperg', 'github-actions', 'leanprover-bot'] |
nobody |
214-75639 7 months ago |
215-64002 7 months ago* |
0-0 0 seconds* |
21611 |
JLimperg author:JLimperg |
Aesop forward benchmark: master no-precomp |
Not a real PR, just for benchmarking. |
merge-conflict |
30/27 |
Mathlib/Data/List/InsertIdx.lean,Mathlib/Tactic/Recall.lean,Mathlib/Topology/List.lean,Test.lean,lake-manifest.json,lakefile.lean,lean-toolchain |
7 |
4 |
['JLimperg', 'github-actions', 'leanprover-bot'] |
nobody |
214-75638 7 months ago |
215-63958 7 months ago* |
0-0 0 seconds* |
21612 |
JLimperg author:JLimperg |
Aesop forward benchmark: master precomp |
Not a real PR, just for benchmarking. |
merge-conflict |
30/27 |
Mathlib/Data/List/InsertIdx.lean,Mathlib/Tactic/Recall.lean,Mathlib/Topology/List.lean,Test.lean,lake-manifest.json,lakefile.lean,lean-toolchain |
7 |
3 |
['JLimperg', 'github-actions', 'leanprover-bot'] |
nobody |
214-75637 7 months ago |
215-63839 7 months ago* |
0-0 0 seconds* |
10678 |
adri326 author:adri326 |
feat(Topology/UniformSpace): prove that a uniform space is completely regular |
Provides the pseudometric definition of a uniform space (for any open set `s` and `x ∈ s`, there exists a finite family of pseudometric spaces on `X` and an `ε > 0`, such that the intersection of the balls of these pseudometric spaces is a subset of `s`),
and uses it to prove that `UniformSpace X` implies `CompletelyRegularSpace X`.
---
This PR aims to close the gap of pi-base's theorem [T345](https://topology.pi-base.org/theorems/T000345), which says that topological groups are completely regular. We already have a proof that topological groups are uniform, but it turns out that we do not have any connection between `UniformSpace X` and `CompletelyRegularSpace X`.
There is an equivalence between `UniformSpace X` and `CompletelyRegularSpace X`: the former implies the latter, and the latter implies *the existence of* the former. This PR provides the first half of this equivalence.
The construction of the pseudometric definition is based on N. Bourbaki, Chapter 9, Theorem 4.1
The proof that a uniform space is completely regular is based on [the outline on mathexchange](https://math.stackexchange.com/questions/494718/how-to-prove-that-every-uniform-space-is-completely-regular).
I tried to outline the major steps of the different proofs inside of comments; I can happily be more verbose to clear up any confusion.
See [the corresponding Zulip discussion](https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/Some.20missing.2C.20accessible.2C.20topology.20results) for more context.
[](https://gitpod.io/from-referrer/)
|
t-topology
merge-conflict
awaiting-author
|
332/0 |
Mathlib.lean,Mathlib/Topology/UniformSpace/Basic.lean,Mathlib/Topology/UniformSpace/CompletelyRegular.lean |
3 |
6 |
['ADedecker', 'adri326'] |
ADedecker assignee:ADedecker |
214-51165 7 months ago |
214-51165 7 months ago |
17-44773 17 days |
20030 |
vihdzp author:vihdzp |
refactor: avoid ordinals in Nöbeling's theorem |
---
[](https://gitpod.io/from-referrer/)
|
t-topology
merge-conflict
WIP
help-wanted
|
356/428 |
Mathlib/Topology/Category/Profinite/Nobeling.lean |
1 |
1 |
['github-actions'] |
nobody |
213-20750 7 months ago |
213-20750 7 months ago |
0-0 0 seconds |
18785 |
erdOne author:erdOne |
feat(CategoryTheory): command that generates instances for `MorphismProperty` |
Co-authored-by: Calle Sönne
---
[](https://gitpod.io/from-referrer/)
|
t-category-theory
t-meta
merge-conflict
awaiting-author
|
369/0 |
Mathlib.lean,Mathlib/CategoryTheory/MorphismProperty/Tactic.lean,MathlibTest/AddMorphismPropertyInstances.lean,scripts/noshake.json |
4 |
19 |
['alexjbest', 'chrisflav', 'erdOne', 'github-actions', 'grunweg', 'jcommelin', 'joelriou'] |
nobody |
212-67675 7 months ago |
212-67675 7 months ago |
52-4682 52 days |
15942 |
grunweg author:grunweg |
chore: move style linters into their own file; document all current linters |
Just to show the overall direction: this PR is just a tracking PR; it is easier to re-do the remaining pieces individually.
- [x] depends on: #19529 (and needs a merge afterwards)
---
The documenting of items should move into Tactic.Linter...
[](https://gitpod.io/from-referrer/)
|
t-linter
merge-conflict
awaiting-author
|
634/287 |
Mathlib.lean,Mathlib/Analysis/SpecialFunctions/BinaryEntropy.lean,Mathlib/Geometry/Manifold/Instances/Real.lean,Mathlib/Init.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Common.lean,Mathlib/Tactic/Linter.lean,Mathlib/Tactic/Linter/AdmitLinter.lean,Mathlib/Tactic/Linter/GlobalAttributeIn.lean,Mathlib/Tactic/Linter/HashCommandLinter.lean,Mathlib/Tactic/Linter/HaveLetLinter.lean,Mathlib/Tactic/Linter/Lint.lean,Mathlib/Tactic/Linter/OldObtain.lean,Mathlib/Tactic/Linter/RefineLinter.lean,Mathlib/Tactic/Linter/Style.lean,Mathlib/Tactic/Linter/UnusedTactic.lean,Mathlib/Util/SleepHeartbeats.lean,lakefile.lean,test/AdmitLinter.lean,test/Change.lean,test/Check.lean,test/Clear!.lean,test/ClearExcept.lean,test/Clear_.lean,test/DefEqTransformations.lean,test/DeriveToExpr.lean,test/ExtractGoal.lean,test/ExtractLets.lean,test/GuardGoalNums.lean,test/GuardHypNums.lean,test/HashCommandLinter.lean,test/Lint.lean,test/LintStyle.lean,test/MfldSetTac.lean,test/MinImports.lean,test/SimpRw.lean,test/SplitIfs.lean,test/TermBeta.lean,test/TypeCheck.lean,test/UnsetOption.lean,test/Use.lean,test/basicTactics.lean,test/casesm.lean,test/convert.lean,test/fail_if_no_progress.lean,test/fun_prop_dev.lean,test/itauto.lean,test/meta.lean,test/notation3.lean,test/recover.lean,test/says.lean,test/symm.lean,test/trace.lean,test/trans.lean |
54 |
5 |
['github-actions', 'grunweg', 'joneugster', 'mathlib4-dependent-issues-bot'] |
nobody |
211-7899 6 months ago |
211-7899 6 months ago |
0-36287 10 hours |
16311 |
madvorak author:madvorak |
feat(Computability): regular languages are context-free |
---
[](https://gitpod.io/from-referrer/)
|
t-computability
merge-conflict
WIP
|
72/0 |
Mathlib.lean,Mathlib/Computability/Chomsky.lean,Mathlib/Computability/ContextFreeGrammar.lean |
3 |
7 |
['Rida-Hamadani', 'YaelDillies', 'github-actions', 'madvorak'] |
nobody |
210-74094 6 months ago |
210-74094 6 months ago |
0-0 0 seconds |
19943 |
AlexLoitzl author:AlexLoitzl |
feat(Computability): Add Chomsky Normal Form Grammar and translation |
- Define Chomsky normal form grammars
- Add language-preserving translation between context-free grammars and Chomsky normal form grammars
Co-authored-by: Martin Dvorak martin.dvorak@matfyz.cz
---
[](https://gitpod.io/from-referrer/)
|
t-computability
new-contributor
merge-conflict
awaiting-author
|
3151/0 |
Mathlib.lean,Mathlib/Computability/ChomskyNormalForm/Basic.lean,Mathlib/Computability/ChomskyNormalForm/EmptyElimination.lean,Mathlib/Computability/ChomskyNormalForm/LengthRestriction.lean,Mathlib/Computability/ChomskyNormalForm/TerminalRestriction.lean,Mathlib/Computability/ChomskyNormalForm/Translation.lean,Mathlib/Computability/ChomskyNormalForm/UnitElimination.lean,Mathlib/Computability/ContextFreeGrammar.lean |
8 |
59 |
['AlexLoitzl', 'YaelDillies', 'github-actions', 'kim-em', 'madvorak'] |
nobody |
210-73847 6 months ago |
210-73847 6 months ago |
37-29014 37 days |
19616 |
adamtopaz author:adamtopaz |
fix: Fix the definition of the absolute Galois group of a field |
Previously it was defined as the Galois group of the algebraic closure, as opposed to the separable closure.
Also, this adds some missing instances for this group.
Still missing is compactness, but that seems like a bigger project.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-number-theory
merge-conflict
awaiting-author
label:t-algebra$ |
23/8 |
Mathlib/FieldTheory/AbsoluteGaloisGroup.lean,Mathlib/FieldTheory/KrullTopology.lean |
2 |
4 |
['acmepjz', 'alreadydone', 'github-actions'] |
nobody |
210-72082 6 months ago |
210-72082 6 months ago |
3-64280 3 days |
17005 |
YnirPaz author:YnirPaz |
feat(SetTheory/Cardinal/Regular): define singular cardinals |
Define singular cardinals and prove basic lemmas about them.
---
[](https://gitpod.io/from-referrer/)
|
t-set-theory
merge-conflict
WIP
|
94/1 |
Mathlib.lean,Mathlib/SetTheory/Cardinal/Regular.lean,Mathlib/SetTheory/Ordinal/Basic.lean |
3 |
28 |
['YaelDillies', 'YnirPaz', 'github-actions', 'vihdzp'] |
nobody |
208-20803 6 months ago |
284-13985 9 months ago |
34-18388 34 days |
18952 |
Command-Master author:Command-Master |
chore: deprecate `Trunc` |
---
[](https://gitpod.io/from-referrer/)
|
t-data
merge-conflict
WIP
|
283/57 |
Mathlib/CategoryTheory/EpiMono.lean,Mathlib/CategoryTheory/Preadditive/Biproducts.lean,Mathlib/Data/DFinsupp/Defs.lean,Mathlib/Data/Fintype/Basic.lean,Mathlib/Data/Fintype/Option.lean,Mathlib/Data/Fintype/Quotient.lean,Mathlib/Data/Quot.lean,Mathlib/Data/Semiquot.lean,Mathlib/GroupTheory/Perm/Cycle/Factors.lean,Mathlib/GroupTheory/Perm/Sign.lean,Mathlib/LinearAlgebra/Determinant.lean,Mathlib/Logic/Equiv/List.lean |
12 |
8 |
['eric-wieser', 'github-actions', 'vihdzp'] |
nobody |
207-58420 6 months ago |
207-58420 6 months ago |
0-0 0 seconds |
18463 |
vihdzp author:vihdzp |
feat(SetTheory/Ordinal/Notation/FundamentalSequence): define type of fundamental sequences |
We define `Sequence α` as the type of sequences with length 0, 1, or `ω`, and give a basic API. A subsequent PR will introduce the notion of a (countable and computable) fundamental sequence and establish basic results.
The goal of this is to generalize [`ONote.fundamentalSequence`](https://leanprover-community.github.io/mathlib4_docs/Mathlib/SetTheory/Ordinal/Notation.html#ONote.fundamentalSequence) to allow the construction of fundamental sequences for other ordinal notations.
---
See [my ordinal notation repository](https://github.com/vihdzp/ordinal-notation/blob/a6fdd7fe7cb521e686ea271902e7e5496f1804d3/OrdinalNotation/Cantor.lean#L1218) for a demonstration of how this API looks in practice.
[](https://gitpod.io/from-referrer/)
|
t-set-theory
t-order
merge-conflict
|
174/1 |
Mathlib.lean,Mathlib/SetTheory/Ordinal/Notation/Cantor.lean,Mathlib/SetTheory/Ordinal/Notation/FundamentalSequence.lean |
3 |
19 |
['YnirPaz', 'b-mehta', 'github-actions', 'vihdzp'] |
nobody |
206-20180 6 months ago |
206-20180 6 months ago |
52-25108 52 days |
12054 |
adomani author:adomani |
feat: auto-bugs |
This PR introduces a linter for suggesting bugs in tactics.
See
* #12077
* #12083
* #12084
for some bugs exposed by the test suite.
---
[](https://gitpod.io/from-referrer/)
|
t-meta
merge-conflict
awaiting-author
|
737/0 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter/MetaTesting.lean,scripts/noshake.json,test/MetaTesting.lean |
5 |
20 |
['adomani', 'eric-wieser', 'github-actions', 'joneugster', 'kim-em'] |
joneugster assignee:joneugster |
205-30275 6 months ago |
205-30275 6 months ago |
45-6057 45 days |
5062 |
adomani author:adomani |
feat(Tactic/Prune + test/Prune): add `prune` tactic, for removing unnecessary hypotheses |
This tactic removes very conservatively all local declarations that
1. do not appear in the main goal,
2. do not appear in a declaration that appears in the main goal,
3. ... and so on recursively.
The main motivation for this tactic is that all available variables in the current `namespace/section` appear in the goal state, not just the ones that are needed for the statement to type-check. Using `prune` mitigates this situation.
The tactic also admits an optional natural number argument: `prune n` removes all variables that have not appeared at the `(n+1)`-st stage in the above list. Thus, `prune 0` only leaves the variables needed for the statement to type-check. Also, for sufficiently large `n`, `prune n` is a synonym for `prune`.
[Zulip discussion](https://leanprover.zulipchat.com/#narrow/stream/270676-lean4/topic/substitute.20for.20.60include.2Fomit.60.3F)
---
[](https://gitpod.io/from-referrer/)
|
t-meta
merge-conflict
modifies-tactic-syntax
awaiting-author
|
181/0 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Prune.lean,test/Prune.lean |
4 |
5 |
['adomani', 'j-loreaux', 'kmill'] |
nobody |
204-83982 6 months ago |
204-83982 6 months ago |
195-56460 195 days |
22169 |
JLimperg author:JLimperg |
Aesop forward benchmark: forward no-precomp naive |
Not a real PR, just for benchmarking. |
merge-conflict |
31/27 |
Mathlib/Data/List/InsertIdx.lean,Mathlib/Tactic/Recall.lean,Mathlib/Topology/List.lean,Test.lean,lake-manifest.json,lakefile.lean,lean-toolchain |
7 |
6 |
['JLimperg', 'github-actions', 'leanprover-bot'] |
nobody |
203-49646 6 months ago |
203-61700 6 months ago* |
0-0 0 seconds* |
21433 |
grunweg author:grunweg |
chore: change more lemmas to be about enorm instead of nnnorm |
---
- [x] depends on: #21782
- [x] depends on: #21783 (and this PR modifies the file split, and file splits are painful to merge over)
[](https://gitpod.io/from-referrer/)
|
carleson
t-measure-probability
merge-conflict
awaiting-author
|
172/71 |
Mathlib/Analysis/Distribution/SchwartzSpace.lean,Mathlib/Analysis/Normed/Group/Basic.lean,Mathlib/Analysis/SpecialFunctions/Pow/NNReal.lean,Mathlib/Data/ENNReal/Basic.lean,Mathlib/MeasureTheory/Function/LpSeminorm/Basic.lean,Mathlib/MeasureTheory/Function/LpSeminorm/CompareExp.lean,Mathlib/MeasureTheory/Function/LpSpace/Basic.lean,Mathlib/MeasureTheory/Function/LpSpace/ContinuousFunctions.lean,Mathlib/MeasureTheory/Function/UniformIntegrable.lean |
9 |
18 |
['RemyDegenne', 'github-actions', 'grunweg', 'j-loreaux', 'mathlib4-dependent-issues-bot'] |
nobody |
203-48835 6 months ago |
205-82319 6 months ago |
2-42743 2 days |
22171 |
JLimperg author:JLimperg |
Aesop forward benchmark: forward no-precomp naive rpinf pr-release |
Not a real PR, just for benchmarking. |
merge-conflict |
31/27 |
Mathlib/Data/List/InsertIdx.lean,Mathlib/Tactic/Recall.lean,Mathlib/Topology/List.lean,Test.lean,lake-manifest.json,lakefile.lean,lean-toolchain |
7 |
5 |
['JLimperg', 'github-actions', 'leanprover-bot'] |
nobody |
202-57519 6 months ago |
203-61263 6 months ago* |
0-0 0 seconds* |
21099 |
chrisflav author:chrisflav |
chore(RingTheory/Generators): use unification hints for variables and relations |
When working with generators and presentations, we rely on the `MvPolynomial` API, but since the type of variables is bundled in `Generators R S`, many lemmas don't apply with `rw` or `simp`, because they can't see through the definition of `vars` in constructions such as `Generators.comp` and `Generators.localizationAway`.
A possible approach is to make all of these constructions `abbrev`s, but this causes `simp` to also unfold `val` which is not always desirable. More generally, it is then harder to predict how instance search and `simp` behave. This approach is tried in #21050, but causes many regressions.
This approach is less invasive, as it uses `unif_hint` to unify the `vars` (and `rels`) fields of constructions with the correct type.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
label:t-algebra$ |
231/91 |
Mathlib/Algebra/Module/Presentation/Differentials.lean,Mathlib/RingTheory/Generators.lean,Mathlib/RingTheory/Kaehler/JacobiZariski.lean,Mathlib/RingTheory/Presentation.lean,Mathlib/RingTheory/Smooth/StandardSmooth.lean |
5 |
16 |
['chrisflav', 'erdOne', 'github-actions', 'leanprover-bot', 'mattrobball'] |
nobody |
201-65416 6 months ago |
201-65416 6 months ago |
27-75210 27 days |
21269 |
CharredLee author:CharredLee |
(WIP) feat (CategoryTheory/Topos): Add topos theory content |
This code contains basic definitions and results in topos theory, including the definition of a subobject classifier, power objects, and topoi. It is proved that every topos has exponential objects, i.e. "internal homs". The mathematical content follows chapter IV sections 1-2 of Mac Lane and Moerdijk's text "Sheaves in Geometry and Logic".
---
- [x] depends on: #21281
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-category-theory
merge-conflict
awaiting-author
WIP
|
1269/0 |
Mathlib.lean,Mathlib/CategoryTheory/Topos/Basic.lean,Mathlib/CategoryTheory/Topos/Classifier.lean,Mathlib/CategoryTheory/Topos/Exponentials.lean,Mathlib/CategoryTheory/Topos/Power.lean |
5 |
10 |
['CharredLee', 'gio256', 'github-actions', 'joelriou', 'mathlib4-dependent-issues-bot'] |
nobody |
200-40119 6 months ago |
200-40119 6 months ago |
0-13879 3 hours |
12394 |
JADekker author:JADekker |
feat : define pre-tight and tight measures |
Define tight measures (by first defining separable and pre-tight measures).
Define some api for all three concepts
Prove Ulam's tightness theorem and a strengthened version of this.
---
[](https://gitpod.io/from-referrer/)
|
t-measure-probability
merge-conflict
please-adopt
awaiting-author
|
503/0 |
Mathlib.lean,Mathlib/MeasureTheory/Measure/Tight.lean |
2 |
34 |
['EtienneC30', 'JADekker', 'github-actions', 'sgouezel'] |
nobody |
199-69012 6 months ago |
199-69012 6 months ago |
2-604 2 days |
20454 |
urkud author:urkud |
chore(TangentCone): review names |
Also add some `@[simp]` attrs.
---
[](https://gitpod.io/from-referrer/)
|
t-analysis
merge-conflict
|
201/139 |
Mathlib/Analysis/Analytic/IteratedFDeriv.lean,Mathlib/Analysis/Calculus/ContDiff/Basic.lean,Mathlib/Analysis/Calculus/ContDiff/Bounds.lean,Mathlib/Analysis/Calculus/ContDiff/Defs.lean,Mathlib/Analysis/Calculus/ContDiff/FTaylorSeries.lean,Mathlib/Analysis/Calculus/Deriv/Abs.lean,Mathlib/Analysis/Calculus/Deriv/Basic.lean,Mathlib/Analysis/Calculus/FDeriv/Add.lean,Mathlib/Analysis/Calculus/FDeriv/Basic.lean,Mathlib/Analysis/Calculus/FDeriv/Equiv.lean,Mathlib/Analysis/Calculus/FDeriv/Measurable.lean,Mathlib/Analysis/Calculus/FDeriv/RestrictScalars.lean,Mathlib/Analysis/Calculus/FDeriv/Symmetric.lean,Mathlib/Analysis/Calculus/IteratedDeriv/Lemmas.lean,Mathlib/Analysis/Calculus/MeanValue.lean,Mathlib/Analysis/Calculus/TangentCone.lean,Mathlib/Analysis/Calculus/Taylor.lean,Mathlib/Analysis/Calculus/VectorField.lean,Mathlib/Analysis/Convex/SpecificFunctions/Deriv.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/InverseDeriv.lean,Mathlib/Geometry/Manifold/Instances/Real.lean,Mathlib/Geometry/Manifold/IsManifold/Basic.lean,Mathlib/Geometry/Manifold/MFDeriv/UniqueDifferential.lean,Mathlib/Geometry/Manifold/VectorBundle/Tangent.lean,Mathlib/MeasureTheory/Integral/FundThmCalculus.lean |
25 |
3 |
['github-actions', 'sgouezel', 'urkud'] |
nobody |
199-9015 6 months ago |
199-9015 6 months ago |
12-11675 12 days |
21608 |
JLimperg author:JLimperg |
Aesop forward benchmark: forward no-precomp rpinf pr-release |
Not a real PR, just for benchmarking. |
merge-conflict |
38/29 |
Mathlib/Data/List/InsertIdx.lean,Mathlib/Data/Nat/Prime/Defs.lean,Mathlib/Tactic/Recall.lean,Mathlib/Topology/List.lean,Test.lean,lake-manifest.json,lakefile.lean,lean-toolchain |
8 |
13 |
['JLimperg', 'github-actions', 'leanprover-bot'] |
nobody |
198-70148 6 months ago |
215-64212 7 months ago* |
0-0 0 seconds* |
21609 |
JLimperg author:JLimperg |
Aesop forward benchmark: forward no-precomp |
Not a real PR, just for benchmarking. |
merge-conflict |
38/29 |
Mathlib/Data/List/InsertIdx.lean,Mathlib/Data/Nat/Prime/Defs.lean,Mathlib/Tactic/Recall.lean,Mathlib/Topology/List.lean,Test.lean,lake-manifest.json,lakefile.lean,lean-toolchain |
8 |
13 |
['JLimperg', 'github-actions', 'leanprover-bot'] |
nobody |
198-68512 6 months ago |
215-64076 7 months ago* |
0-0 0 seconds* |
16550 |
awainverse author:awainverse |
feat(ModelTheory): A typeclass for languages expanding other languages |
Defines `L.Expands L'` to consist of a privileged injective inclusion, `L'.Inclusion L`, from `L'` to `L`, corresponding to one language being a subset of the other in set-theoretic foundations.
Replaces `L.IsOrdered` with `L.Expands Language.order` and `L.OrderLHom` with `Language.order.Inclusion L`
Redefines `leSymb` in terms of `Language.order.Inclusion L`
Deletions:
- `FirstOrder.Language.IsOrdered`
- `FirstOrder.Language.OrderLHom`
- `instance : IsOrdered Language.order`
- `sum.instIsOrdered`
---
[](https://gitpod.io/from-referrer/)
|
t-logic
merge-conflict
awaiting-author
|
97/43 |
Mathlib/ModelTheory/LanguageMap.lean,Mathlib/ModelTheory/Order.lean |
2 |
9 |
['YaelDillies', 'awainverse', 'github-actions'] |
nobody |
198-47883 6 months ago |
198-47884 6 months ago |
0-61590 17 hours |
13686 |
fpvandoorn author:fpvandoorn |
feat: some finset lemmas |
* From the Sobolev inequality project
* The increase in imports in `Mathlib.Data.Finset.Update` is not problematic: it is only imported in MeasureTheory files.
Co-authored-by: Heather Macbeth 25316162+hrmacbeth@users.noreply.github.com
---
[](https://gitpod.io/from-referrer/)
|
t-data
merge-conflict
awaiting-author
|
69/7 |
Mathlib/Data/Finset/Basic.lean,Mathlib/Data/Finset/Lattice/Lemmas.lean,Mathlib/Data/Finset/Update.lean |
3 |
7 |
['YaelDillies', 'fpvandoorn', 'github-actions', 'urkud'] |
nobody |
197-47514 6 months ago |
197-47514 6 months ago |
98-49006 98 days |
14313 |
grhkm21 author:grhkm21 |
feat(RepresentationTheory/FdRep): FdRep is a full subcategory of Rep |
```
/-- Equivalence between `FDRep` and the full subcategory of finite dimensional `Rep`. -/
def equivFiniteDimensional :
FDRep k G ≌ FullSubcategory (fun V : Rep k G ↦ FiniteDimensional k V)
``` |
new-contributor
t-algebra
t-category-theory
merge-conflict
label:t-algebra$ |
47/8 |
Mathlib/RepresentationTheory/FDRep.lean |
1 |
19 |
['github-actions', 'grhkm21', 'joelriou', 'kim-em', 'mathlib-bors'] |
nobody |
196-82445 6 months ago |
196-82445 6 months ago |
125-12755 125 days |
18626 |
hannahfechtner author:hannahfechtner |
feat : define Artin braid groups |
Define the Artin braid group on infinitely many strands. Includes a toGroup function which defines a function out of the braid group to any other group (given a function which satisfies the braid relations)
(more to come in this file; next up: Artin braid groups on finitely many strands)
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-algebra
merge-conflict
awaiting-author
label:t-algebra$ |
91/0 |
Mathlib.lean,Mathlib/GroupTheory/SpecificGroups/BraidGroup/Basic.lean |
2 |
22 |
['github-actions', 'hannahfechtner', 'jcommelin', 'joelriou'] |
nobody |
195-66756 6 months ago |
195-66756 6 months ago |
15-40648 15 days |
10823 |
alexkeizer author:alexkeizer |
feat: convert curried type functions into uncurried type functions |
Adds a conversion `TypeFun.ofCurried : CurriedTypeFun.{u, v} n -> TypeFun.{u, v} n`,
where `CurriedTypeFun.{u,v} n` is a (def-eq) abbreviation for `Type u -> ... -> Type u -> Type v`, i.e., the type of *curried* functions taking `n` arguments of type `Type u` to return an element of `Type v`, and
`TypeFun.{u, v} n` is an abbreviation for `TypeVec.{u} n -> Type v`.
It is generally more idiomatic to define type functions with multiple arguments in the curried style, but in the QPF development we use the uncurried equivalent `TypeVec n -> Type _`. Thus, having a canonical conversion from curried functions to uncurried gives us a canonical way to ask if a curried type function, say `Sum` is a QPF (namely, "is there an instance of `MvQPF (TypeFun.ofCurried Sum)`").
---
This is code ported from https://github.com/alexkeizer/QpfTypes, where this conversion is crucial in presenting a high-level interface, in terms of idiomatic, curried, type functions to users, while being built on QPFs (and thus, uncurried typefunctions) underneath.
There is also a conversion in the other direction, from uncurried to curried, which I've decided to PR later, to keep this PR smaller and hopefully easier to review.
- [x] depends on: #10818 (all changes to `Fin2.lean` are part of 10818, not the current PR)
[](https://gitpod.io/from-referrer/)
|
t-data
merge-conflict
awaiting-author
|
66/0 |
Mathlib.lean,Mathlib/Data/TypeFun.lean |
2 |
9 |
['YaelDillies', 'alexkeizer', 'github-actions', 'leanprover-community-mathlib4-bot'] |
nobody |
195-60476 6 months ago |
unknown |
unknown |
13648 |
urkud author:urkud |
feat(Topology/Module): generalize `ContinuousLinearMap.compSL` |
Generalize `ContinuousLinearMap.compSL` to topological vector spaces.
---
- [ ] depends on: #15217
This PR is not polished yet, but the main statement is there.
@ADedecker This answers a question I asked you on Zulip a few months ago.
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-analysis
t-topology
merge-conflict
awaiting-author
label:t-algebra$ |
23/18 |
Mathlib/Analysis/NormedSpace/OperatorNorm/Bilinear.lean,Mathlib/Topology/Algebra/Module/StrongTopology.lean |
2 |
5 |
['fpvandoorn', 'github-actions', 'mathlib4-dependent-issues-bot', 'urkud'] |
nobody |
193-83566 6 months ago |
193-83566 6 months ago |
0-0 0 seconds |
21684 |
mattrobball author:mattrobball |
draft |
|
merge-conflict |
13/11 |
Mathlib/CategoryTheory/Category/Cat/AsSmall.lean,Mathlib/CategoryTheory/Closed/FunctorToTypes.lean,Mathlib/CategoryTheory/Closed/Types.lean,Mathlib/FieldTheory/IsAlgClosed/Classification.lean,Mathlib/SetTheory/Ordinal/Basic.lean,Mathlib/Topology/Category/LightProfinite/Basic.lean,lean-toolchain |
7 |
4 |
['github-actions', 'leanprover-bot', 'mattrobball'] |
nobody |
193-77136 6 months ago |
193-77136 6 months ago |
0-0 0 seconds |
21722 |
mattrobball author:mattrobball |
test |
|
merge-conflict |
76/23 |
Mathlib/CategoryTheory/Category/Cat/AsSmall.lean,Mathlib/CategoryTheory/Closed/FunctorToTypes.lean,Mathlib/CategoryTheory/Closed/Types.lean,Mathlib/FieldTheory/IsAlgClosed/Classification.lean,Mathlib/Order/Hom/Lattice.lean,Mathlib/SetTheory/Ordinal/Basic.lean,Mathlib/Topology/Category/LightProfinite/Basic.lean,lean-toolchain,scratch.lean |
9 |
4 |
['github-actions', 'leanprover-bot', 'mattrobball'] |
nobody |
193-77135 6 months ago |
193-77135 6 months ago |
0-0 0 seconds |
22408 |
JLimperg author:JLimperg |
Aesop forward bench: precomp only rpinf |
---
Not a real PR (yet), just for benchmarking.
[](https://gitpod.io/from-referrer/)
|
dependency-bump
merge-conflict
|
5/3 |
lake-manifest.json,lakefile.lean,scripts/bench/fake-root/lib/lean/libleanshared.so,scripts/bench/run |
4 |
6 |
['JLimperg', 'github-actions', 'leanprover-bot'] |
nobody |
193-71970 6 months ago |
193-71970 6 months ago |
0-0 0 seconds |
21339 |
vihdzp author:vihdzp |
fix(Data/List/Lex): remove duplicate `List.LE` instance |
Mathlib currently duplicates the Lean core instance for `≤` in lists in an incompatible way. We delete this duplicate instance.
See [Zulip](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Two.20.60List.2ELE.60.20instances.3F/near/497241115).
---
This is a very quick and dirty fix. Core Lean provides all of the theorems we need to prove `≤` forms a linear order, but it provides them in terms of `Std` relation typeclasses which currently see no use in Mathlib. I've added the instances that were required to get the list theorems working. In the future, we really ought to unify the core and Mathlib relation typeclasses.
[](https://gitpod.io/from-referrer/)
|
t-data
merge-conflict
|
24/22 |
Mathlib/Data/List/Lex.lean,Mathlib/Data/String/Basic.lean,Mathlib/Topology/Category/Profinite/Nobeling.lean |
3 |
1 |
['github-actions'] |
nobody |
193-64308 6 months ago |
193-64308 6 months ago |
16-65973 16 days |
16837 |
vihdzp author:vihdzp |
feat(Data/List/SplitBy): characterization of `List.splitBy` |
---
- [x] depends on: #16818
[](https://gitpod.io/from-referrer/)
|
t-data
merge-conflict
awaiting-author
|
151/9 |
Mathlib/Data/List/Flatten.lean,Mathlib/Data/List/SplitBy.lean |
2 |
13 |
['YaelDillies', 'github-actions', 'mathlib4-dependent-issues-bot', 'vihdzp'] |
nobody |
193-24623 6 months ago |
193-24623 6 months ago |
9-85039 9 days |
16421 |
FR-vdash-bot author:FR-vdash-bot |
feat: `QuotLike` |
This typeclass is primarily for use by type synonyms of `Quot` and `Quotient`. Using `QuotLike` API for type synonyms of `Quot` and `Quotient` will avoid defeq abuse caused by directly using `Quot` and `Quotient` APIs.
---
Some of the naming may need to be discussed. For example, `⟦·⟧` is currently called `mkQ` in names. This distinguishes it from other `.mk`s and makes it possible to write the quotient map as `mkQ` `mkQ'` `mkQ_ h`. But this will also require changing the old lemma names.
[Zulip](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/migrate.20to.20.60QuotLike.60.20API)
[](https://gitpod.io/from-referrer/)
|
t-data
RFC
merge-conflict
awaiting-author
|
735/1 |
Mathlib.lean,Mathlib/Data/QuotLike.lean,Mathlib/Logic/Relation.lean,test/QuotLike.lean |
4 |
7 |
['FR-vdash-bot', 'YaelDillies', 'github-actions', 'urkud'] |
nobody |
193-24623 6 months ago |
193-24623 6 months ago |
58-8650 58 days |
19700 |
vihdzp author:vihdzp |
chore(SetTheory/Ordinal/Basic): tweak `type r = 0`, `type r = 1`, etc. lemmas |
We give shorter names to these lemmas (e.g. `type_eq_zero` instead of `type_eq_zero_of_empty`), and deprecate a bunch of duplicates.
---
[](https://gitpod.io/from-referrer/)
|
t-set-theory
awaiting-CI
merge-conflict
|
51/38 |
Mathlib/SetTheory/Ordinal/Basic.lean |
1 |
1 |
['github-actions'] |
nobody |
193-24376 6 months ago |
193-24376 6 months ago |
0-0 0 seconds |
21959 |
BGuillemet author:BGuillemet |
feat(Topology/ContinuousMap): Stone-Weierstrass theorem for MvPolynomial |
Add the subalgebra of multivariate polynomials and prove it separates points, on the same model as `ContinuousMap/Polynomial.lean`.
Prove the Stone-Weierstrass theorem and some variations for multivariate polynomials.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-topology
merge-conflict
|
285/1 |
Mathlib.lean,Mathlib/Topology/ContinuousMap/MvPolynomial.lean,Mathlib/Topology/ContinuousMap/StoneWeierstrass.lean |
3 |
1 |
['github-actions'] |
nobody |
191-68459 6 months ago |
191-68459 6 months ago |
16-76141 16 days |
19177 |
adomani author:adomani |
test: the findDefEqAbuse linter |
This is a prototype, as per [this Zulip discussion](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Locating.20defeq.20abuse)
---
[](https://gitpod.io/from-referrer/)
|
large-import
merge-conflict
|
126/0 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter.lean,Mathlib/Tactic/Linter/FindDefEqAbuse.lean,MathlibTest/FindDefEqAbuse.lean |
5 |
1 |
['github-actions'] |
nobody |
189-70472 6 months ago |
189-70472 6 months ago |
0-0 0 seconds |
20750 |
adomani author:adomani |
feat: the envLinter syntax linter |
The `envLinter` syntax linter emits a warning at the end of a file if `#lint` reports an error.
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-linter
merge-conflict
|
69/0 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter.lean,Mathlib/Tactic/Linter/EnvLinter.lean,MathlibTest/EnvLinter.lean |
5 |
15 |
['adomani', 'github-actions', 'grunweg'] |
nobody |
189-70226 6 months ago |
189-70226 6 months ago |
51-71438 51 days |
22359 |
adomani author:adomani |
feat(whitespace): do not allow indented doc-strings |
In a doc-string, Do not allow the first character after the first line break to be a space.
---
There are approximately 2.5k exceptions. I think that they should be unindented, judging from the sample that I looked at, but won't act on it, unless there is a clear plan to fix and merge this modification!
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-linter
merge-conflict
WIP
|
222/70 |
Archive/Wiedijk100Theorems/BuffonsNeedle.lean,Mathlib.lean,Mathlib/Algebra/Module/SpanRank.lean,Mathlib/AlgebraicTopology/SimplicialSet/NerveAdjunction.lean,Mathlib/Analysis/Asymptotics/ExpGrowth.lean,Mathlib/Data/Matroid/Circuit.lean,Mathlib/Init.lean,Mathlib/Lean/Meta/RefinedDiscrTree/Encode.lean,Mathlib/LinearAlgebra/Dimension/StrongRankCondition.lean,Mathlib/LinearAlgebra/LinearIndependent/Basic.lean,Mathlib/LinearAlgebra/LinearIndependent/Defs.lean,Mathlib/Tactic.lean,Mathlib/Tactic/FunProp/Decl.lean,Mathlib/Tactic/FunProp/Theorems.lean,Mathlib/Tactic/Linter.lean,Mathlib/Tactic/Linter/DocString.lean,Mathlib/Topology/Path.lean,Mathlib/Topology/UnitInterval.lean,MathlibTest/LintDocstring.lean,lakefile.lean |
20 |
1 |
['github-actions'] |
nobody |
189-69391 6 months ago |
189-69391 6 months ago |
0-0 0 seconds |
18470 |
FR-vdash-bot author:FR-vdash-bot |
perf: lower the priority of `Normed*.to*` instances |
---
From #7873.
[](https://gitpod.io/from-referrer/)
|
slow-typeclass-synthesis
t-algebra
t-analysis
merge-conflict
label:t-algebra$ |
28/0 |
Mathlib/Analysis/Normed/Field/Basic.lean,Mathlib/Analysis/Normed/Group/Basic.lean |
2 |
9 |
['FR-vdash-bot', 'github-actions', 'jcommelin', 'leanprover-bot'] |
nobody |
187-39886 6 months ago |
187-39886 6 months ago |
130-5197 130 days |
16944 |
YnirPaz author:YnirPaz |
feat(SetTheory/Cardinal/Cofinality): lemmas about limit ordinals and cofinality |
Prove that a singular cardinal has a limit aleph index and that a limit ordinal and positive cofinality.
---
[](https://gitpod.io/from-referrer/)
|
t-set-theory
merge-conflict
WIP
|
18/0 |
Mathlib/SetTheory/Cardinal/Cofinality.lean |
1 |
8 |
['YnirPaz', 'github-actions', 'vihdzp'] |
nobody |
186-32762 6 months ago |
186-32762 6 months ago |
1-84890 1 day |
17368 |
Felix-Weilacher author:Felix-Weilacher |
feat(Topology/Baire/BaireMeasurable): add the Kuratowski-Ulam theorem |
Add the Kuratowski-Ulam theorem, which one can think of as a "Fubini" for Baire category.
---
[](https://gitpod.io/from-referrer/)
|
t-topology
merge-conflict
|
187/1 |
Mathlib/MeasureTheory/MeasurableSpace/Basic.lean,Mathlib/Order/Filter/Basic.lean,Mathlib/Topology/Baire/BaireMeasurable.lean,Mathlib/Topology/Constructions.lean,Mathlib/Topology/GDelta/Basic.lean |
5 |
6 |
['Felix-Weilacher', 'github-actions', 'urkud'] |
nobody |
185-63955 6 months ago |
185-63955 6 months ago |
72-13986 72 days |
8767 |
eric-wieser author:eric-wieser |
refactor(Cache): tidy lake-manifest parsing in Cache |
This now respects local copies of Mathlib dependencies (though in practice these invalidate the *online* cache because to point to local copies of Mathlib, the hash for `lakefile.lean` and `lake-manifest.json` is first invalidated).
---
- [x] depends on: #11492
[](https://gitpod.io/from-referrer/)
|
t-meta
merge-conflict
|
49/49 |
Cache/Hashing.lean,Cache/IO.lean,lake-manifest.json |
3 |
8 |
['digama0', 'eric-wieser', 'github-actions', 'leanprover-community-mathlib4-bot'] |
nobody |
184-39618 6 months ago |
366-5568 1 year ago |
119-35643 119 days |
22434 |
qawbecrdtey author:qawbecrdtey |
feat(Mathlib/Analysis/Normed/Lp/WithLp): Added more instances for `WithLp` |
---
[](https://gitpod.io/from-referrer/)
|
t-analysis
merge-conflict
awaiting-author
|
51/22 |
Mathlib/Analysis/Normed/Lp/WithLp.lean |
1 |
11 |
['eric-wieser', 'github-actions', 'leanprover-bot', 'qawbecrdtey'] |
nobody |
183-69057 5 months ago |
183-69057 5 months ago |
1-79072 1 day |
15578 |
znssong author:znssong |
feat(Function): Fixed points of function `f` with `f(x) >= x` |
We added some lemmas of fixed points of function `f` with `f(x) >= x`, where `f : α → α` is a function on a finite type `α`. This will be needed in proof of Bondy-Chvátal theorem.
---
See also branch `meow-sister/BondyChvatal`.
[](https://gitpod.io/from-referrer/) |
new-contributor
t-analysis
merge-conflict
awaiting-author
|
82/0 |
Mathlib.lean,Mathlib/Dynamics/FixedPoints/Basic.lean,Mathlib/Dynamics/FixedPoints/Increasing.lean |
3 |
32 |
['Ruben-VandeVelde', 'YaelDillies', 'github-actions', 'urkud', 'vihdzp', 'znssong'] |
nobody |
183-64285 5 months ago |
183-64285 5 months ago |
29-48368 29 days |
22805 |
ScottCarnahan author:ScottCarnahan |
feat (FieldTheory/Finite): fixed points of frobenius |
This PR identifies the prime field with the fixed points of frobenius.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
WIP
label:t-algebra$ |
325/7 |
Mathlib/Algebra/Algebra/ZMod.lean,Mathlib/Algebra/Field/Subfield/Basic.lean,Mathlib/FieldTheory/Finite/Basic.lean,Mathlib/FieldTheory/Finite/GaloisField.lean |
4 |
1 |
['github-actions'] |
nobody |
181-74997 5 months ago |
181-74997 5 months ago |
0-0 0 seconds |
22660 |
Ruben-VandeVelde author:Ruben-VandeVelde |
chore: follow naming convention around Group.IsNilpotent |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
label:t-algebra$ |
133/67 |
Mathlib/GroupTheory/Frattini.lean,Mathlib/GroupTheory/Nilpotent.lean,Mathlib/GroupTheory/SpecificGroups/ZGroup.lean |
3 |
1 |
['github-actions'] |
nobody |
180-4314 5 months ago |
180-4314 5 months ago |
10-48025 10 days |
13999 |
adomani author:adomani |
feat: a linter to flag potential confusing conventions |
Currently, the linter flags all uses of
* `a - b` where `a b : Nat`;
* `a / b` where `a b : Nat` or `a b : Int`;
* `a / 0` more or less whenever the type of `a` has a `0` and a division.
This comes up often when starting to use Lean and hopefully the flag can help mitigate initial confusions.
When the local context contains the relevant inequality/divisibility hypothesis, the linter is quiet.
A recent [Zulip discussion](https://leanprover.zulipchat.com/#narrow/stream/113489-new-members/topic/not.20understanding.20deliberate.20error.20with.20.60ring.60.20over.20.E2.84.95/near/445879310)
---
To make sure that the linter does not produce errors, #14007 activates the linter on "all" of mathlib. The expectation is that no error is thrown, just warnings.
[](https://gitpod.io/from-referrer/)
|
t-linter
merge-conflict
awaiting-author
|
251/0 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter/Papercut.lean,MathlibTest/Papercut.lean |
4 |
24 |
['Julian', 'YaelDillies', 'adomani', 'eric-wieser', 'github-actions'] |
nobody |
179-36348 5 months ago |
179-36348 5 months ago |
7-47472 7 days |
15991 |
vihdzp author:vihdzp |
feat(SetTheory/Ordinal/CantorNormalForm): alternate CNF recursion principle |
The idea of this recursion principle is that you can build an ordinal by adding one power of `b` at a time, as long as `1 < b ≤ ω`.
---
[](https://gitpod.io/from-referrer/)
|
t-set-theory
t-logic
merge-conflict
awaiting-author
|
43/0 |
Mathlib/SetTheory/Ordinal/Arithmetic.lean,Mathlib/SetTheory/Ordinal/CantorNormalForm.lean,Mathlib/SetTheory/Ordinal/Exponential.lean |
3 |
8 |
['YaelDillies', 'eric-wieser', 'github-actions', 'vihdzp'] |
nobody |
178-84532 5 months ago |
178-84532 5 months ago |
91-50443 91 days |
19698 |
vihdzp author:vihdzp |
refactor(SetTheory/Cardinal/Cofinality): redefine `Order.cof` |
We redefine `Order.cof` as a function on preorders, rather than one well-ordered relations. This allows us to use the `IsCofinal` API, alongside all the other goodies that come from a proper order structure.
Finally, we clean up the `Ordinal.cof` API by relying on order results, rather than trying to haphazardly treat ordinals as sets.
---
- [ ] depends on: #21972
[](https://gitpod.io/from-referrer/)
|
t-set-theory
merge-conflict
WIP
|
502/583 |
Mathlib/Order/Cofinal.lean,Mathlib/SetTheory/Cardinal/Basic.lean,Mathlib/SetTheory/Cardinal/Cofinality.lean,Mathlib/SetTheory/Ordinal/Basic.lean |
4 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
178-82072 5 months ago |
178-82072 5 months ago |
0-0 0 seconds |
20967 |
joneugster author:joneugster |
tracking(CategoryTheory/Enriched/Limits): add conical limits |
Tracking PR for adding conical limits
Co-authored-by: Emily Riehl
Co-authored-by: Dagur Asgeirsson
---
- [x] depends on: #20904
- [x] depends on: #20907
- [x] depends on: #20959
- [x] depends on: #20963
- [x] depends on: #20964
- [x] depends on: #20965
- content source: emilyriehl/infinity-cosmos#78
New implementation (not reflected on this branch yet):
- [x] depends on: #22917
- [x] depends on: #22921
- [ ] depends on: #22923
- [ ] depends on: #22924
[](https://gitpod.io/from-referrer/)
|
infinity-cosmos
t-category-theory
merge-conflict
WIP
|
619/1 |
Mathlib.lean,Mathlib/CategoryTheory/Enriched/Limits/HasConicalLimits.lean,Mathlib/CategoryTheory/Enriched/Limits/HasConicalProducts.lean,Mathlib/CategoryTheory/Enriched/Limits/HasConicalPullbacks.lean,Mathlib/CategoryTheory/Enriched/Limits/HasConicalTerminal.lean,Mathlib/CategoryTheory/Enriched/Limits/IsConicalLimit.lean,Mathlib/CategoryTheory/Enriched/Limits/IsConicalTerminal.lean,Mathlib/CategoryTheory/Enriched/Ordinary/Basic.lean |
8 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
178-41954 5 months ago |
178-41956 5 months ago |
0-0 0 seconds |
19013 |
quangvdao author:quangvdao |
feat(Algebra/BigOperators/Fin): Add `finSigmaFinEquiv` |
This PR adds `finSigmaFinEquiv` which is the equivalence `(i : Fin m) × Fin (n i) ≃ Fin (∑ i, n i)`. This is the dependent version of `finProdFinEquiv`.
CI should be passing, but there are two things I'd like feedback on:
1. When defining the mappings, I have to consider `m = 0` separately. Is there a more uniform definition?
2. I'm proving this as a step toward defining `Fin.join`, which is the analogue of `List.join`. I can now technically define `Fin.join` as:
```
variable {a : Fin n → ℕ} {α : (i : Fin n) → (j : Fin (a i)) → Sort*}
def join (v : (i : Fin n) → (j : Fin (a i)) → α i j) (k : Fin (∑ i, a i)) :
α (finSigmaFinEquiv.invFun k).1 (finSigmaFinEquiv.invFun k).2 :=
v (finSigmaFinEquiv.invFun k).1 (finSigmaFinEquiv.invFun k).2
```
but this looks horrible. This highly motivates refactoring `invFun` as two new definitions:
```
def func1 {n : ℕ} (a : Fin n → ℕ) (k : Fin (∑ i, a i)) : Fin n := sorry
def func2 {n : ℕ} (a : Fin n → ℕ) (k : Fin (∑ i, a i)) : Fin (a (func1 a k)) := sorry
```
I'm not sure what to call these functions. The analogues in the non-dependent case are `divNat` and `modNat`.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
awaiting-author
label:t-algebra$ |
92/16 |
Mathlib/Algebra/BigOperators/Fin.lean |
1 |
14 |
['YaelDillies', 'eric-wieser', 'github-actions', 'quangvdao'] |
nobody |
177-58381 5 months ago |
177-58381 5 months ago |
3-28829 3 days |
20389 |
eric-wieser author:eric-wieser |
feat: generalize results to `WithLp 0` |
---
[](https://gitpod.io/from-referrer/)
|
t-analysis
merge-conflict
|
116/53 |
Mathlib/Analysis/Normed/Lp/PiLp.lean |
1 |
1 |
['github-actions'] |
nobody |
176-46929 5 months ago |
176-46929 5 months ago |
0-0 0 seconds |
19189 |
YnirPaz author:YnirPaz |
feat(SetTheory/Ordinal/Arithmetic): order isomorphism between omega and the natural numbers |
---
[](https://gitpod.io/from-referrer/)
|
t-set-theory
merge-conflict
awaiting-author
|
44/0 |
Mathlib/Order/SuccPred/Limit.lean,Mathlib/SetTheory/Ordinal/Arithmetic.lean |
2 |
21 |
['YaelDillies', 'YnirPaz', 'github-actions', 'vihdzp'] |
nobody |
176-28014 5 months ago |
176-28014 5 months ago |
47-37012 47 days |
19227 |
adomani author:adomani |
fix(CI): unwrap `lake test` in problem matcher |
... and also add a `#guard_msgs` in `AssertImported` test, so that `lake test` properly fails.
[Zulip discussion](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/CI.3A.20noisy.20.22test.20mathlib.22/near/483126955)
---
[](https://gitpod.io/from-referrer/)
|
CI
merge-conflict
awaiting-author
|
9/20 |
.github/build.in.yml,.github/workflows/bors.yml,.github/workflows/build.yml,.github/workflows/build_fork.yml,MathlibTest/AssertImported.lean |
5 |
2 |
['bryangingechen', 'github-actions'] |
nobody |
174-77417 5 months ago |
174-77418 5 months ago |
22-71271 22 days |
20874 |
grunweg author:grunweg |
chore(nolint.yml): use shallow clones |
This should be sufficient, and be slightly faster on CI.
---
[](https://gitpod.io/from-referrer/)
|
CI
merge-conflict
awaiting-author
|
0/3 |
.github/workflows/nolints.yml |
1 |
2 |
['bryangingechen', 'github-actions'] |
nobody |
174-77172 5 months ago |
174-77172 5 months ago |
0-15573 4 hours |
15774 |
kkytola author:kkytola |
feat: Topology on `ENat` |
This PR may contain some results that are not in the PR that adds a toppology on `ENat`.
---
The immediate motivation is to be able to make the right continuity statement of the extended floor function on `ENNReal`, when this floor function is made `ENat`valued as suggested in the PR review of #15269.
The API here is modelled on the early parts of [the corresponding ENNReal file](https://leanprover-community.github.io/mathlib4_docs/Mathlib/Topology/Instances/ENNReal.html#top), although much of this case is more trivial.
- [x] depends on: #15380
[](https://gitpod.io/from-referrer/)
|
t-order
t-topology
merge-conflict
WIP
|
161/9 |
Mathlib/Data/ENat/Basic.lean,Mathlib/Topology/Instances/ENat.lean |
2 |
4 |
['YaelDillies', 'github-actions', 'leanprover-community-mathlib4-bot'] |
nobody |
170-34949 5 months ago |
170-34949 5 months ago |
0-6819 1 hour |
18284 |
chrisflav author:chrisflav |
feat(AlgebraicGeometry): relative gluing of schemes |
We show https://stacks.math.columbia.edu/tag/01LH using #14208. This shall be used to construct the relative spectrum of a quasi-coherent algebra.
---
- [ ] depends on: #14208
[](https://gitpod.io/from-referrer/)
|
t-algebraic-geometry
merge-conflict
WIP
|
1393/7 |
Mathlib.lean,Mathlib/AlgebraicGeometry/Gluing.lean,Mathlib/AlgebraicGeometry/OpenImmersion.lean,Mathlib/AlgebraicGeometry/RelativeGluing.lean,Mathlib/AlgebraicGeometry/Sites/Representability.lean,Mathlib/CategoryTheory/Functor/FullyFaithful.lean,Mathlib/CategoryTheory/Limits/Shapes/Types.lean,Mathlib/CategoryTheory/MorphismProperty/Representable.lean |
8 |
n/a |
['github-actions', 'joelriou', 'mathlib4-dependent-issues-bot'] |
nobody |
169-57701 5 months ago |
unknown |
unknown |
16810 |
urkud author:urkud |
feat: define `(a : ENat) ^ (b : ENat)` |
The definition agrees with `Cardinal.toENat`, i.e., `#(α → β) = #β ^ #α`,
where `#` is the not-yet-defined `ENat.card α = Cardinal.toENat (Cardinal.mk α)`.
---
[](https://gitpod.io/from-referrer/)
|
t-set-theory
t-data
merge-conflict
|
51/0 |
Mathlib.lean,Mathlib/Data/ENat/Pow.lean |
2 |
1 |
['github-actions'] |
nobody |
169-14142 5 months ago |
169-14142 5 months ago |
0-0 0 seconds |
16009 |
Command-Master author:Command-Master |
acyclic graph |
---
[](https://gitpod.io/from-referrer/)
|
t-combinatorics
merge-conflict
WIP
|
232/0 |
Mathlib/Combinatorics/SimpleGraph/Acyclic.lean |
1 |
1 |
['github-actions'] |
nobody |
168-69498 5 months ago |
168-69498 5 months ago |
0-0 0 seconds |
20613 |
grunweg author:grunweg |
chore: golf using `List.toArrayMap` |
---
Depends on batteries#1090 landing in mathlib.
[](https://gitpod.io/from-referrer/)
|
large-import
merge-conflict
|
27/21 |
Cache/Main.lean,Cache/Requests.lean,Mathlib/Lean/Meta/RefinedDiscrTree/Lookup.lean,Mathlib/Tactic/DeriveTraversable.lean,Mathlib/Tactic/Linter/TextBased.lean,Mathlib/Tactic/MoveAdd.lean,Mathlib/Tactic/ToAdditive/Frontend.lean,Mathlib/Util/CompileInductive.lean,Mathlib/Util/GetAllModules.lean,Mathlib/Util/Notation3.lean,scripts/autolabel.lean |
11 |
2 |
['github-actions', 'vihdzp'] |
nobody |
166-33915 5 months ago |
166-33915 5 months ago |
22-82622 22 days |
15989 |
vihdzp author:vihdzp |
feat(SetTheory/Ordinal/Principal): golf theorems on additively principal ordinals |
We add some new results on additively principal ordinals and use them to simplify existing theorems.
---
- [x] depends on: #15990
- [x] depends on: #17740
- [x] depends on: #17741
- [x] depends on: #17742
- [x] depends on: #17842
- [x] depends on: #18902
[](https://gitpod.io/from-referrer/)
|
t-set-theory
t-logic
merge-conflict
awaiting-author
|
64/59 |
Mathlib/SetTheory/Ordinal/Arithmetic.lean,Mathlib/SetTheory/Ordinal/Notation.lean,Mathlib/SetTheory/Ordinal/Principal.lean |
3 |
8 |
['YaelDillies', 'github-actions', 'kbuzzard', 'mathlib4-dependent-issues-bot', 'vihdzp'] |
nobody |
165-25758 5 months ago |
165-25758 5 months ago |
60-46576 60 days |
22682 |
grunweg author:grunweg |
chore(Topology/Homeomorph): split out various constructions |
This makes `Homeomorph.lean` slightly more manageable, and also is a mild import reduction.
edit: also split out IsHomeomorph, as this allows removing the dependencies on Constructions. Let's see if this gains much
---
I don't feel strongly about this PR, but we might as well take it.
- [ ] depends on: #22681
- [ ] depends on #22827
[](https://gitpod.io/from-referrer/)
|
tech debt
t-topology
RFC
merge-conflict
|
341/290 |
Mathlib.lean,Mathlib/Topology/Category/TopCat/ULift.lean,Mathlib/Topology/Homeomorph/Constructions.lean,Mathlib/Topology/Homeomorph/IsHomeomorph.lean,Mathlib/Topology/Homeomorph/Lemmas.lean,Mathlib/Topology/NoetherianSpace.lean |
6 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
165-23521 5 months ago |
165-23521 5 months ago |
14-35834 14 days |
21018 |
markimunro author:markimunro |
feat(Data/Matrix): add file with key definitions and theorems about elementary row operations |
Prove that each elementary row operation is equivalent to a multiplication by an elementary matrix, has another row operation which inverts it, and that each elementary matrix has a left inverse.
This is a very large PR and I understand it will take time. This is my first one and will likely have issues but I will be ready to answer questions/fix them as soon as possible.
Co-authored-by: Christopher Lynch
---
[](https://gitpod.io/from-referrer/)
|
t-data
new-contributor
merge-conflict
awaiting-author
enhancement
|
1230/0 |
Mathlib.lean,Mathlib/Data/Matrix/ElementaryRowOperations.lean,Mathlib/Data/Matrix/GaussianElimination.lean,Mathlib/Data/Matrix/GaussianEliminationOld,Mathlib/Data/Matrix/oldnames,et --hard 18533caba32,lean-toolchain |
7 |
n/a |
['chrisflav', 'eric-wieser', 'github-actions', 'j-loreaux', 'markimunro'] |
nobody |
165-13284 5 months ago |
unknown |
unknown |
23514 |
eric-wieser author:eric-wieser |
refactor: smooth over Lattice/LinearOrder inheritance |
This fixes the forgetful inheritance in `CompleteLinearOrder` and `ConditionallyCompleteLinearOrder`, which previously did not carry `compare` fields. (edit: moved to #23515)
The following is the inheritance diagram before, where the dotted lines are manual instances. Note that every lattice typeclass that extends `LinearOrder` has to implement another dotted line edge, and remember to copy all the necessary data fields.
```mermaid
graph TD
LinearOrder --> Min,Max;
LinearOrder --> PartialOrder;
Lattice --> PartialOrder;
CompleteLinearOrder --> Lattice;
ConditionallyCompleteLinearOrder --> Lattice;
LinearOrder-.-> Lattice;
CompleteLinearOrder -.-> LinearOrder;
ConditionallyCompleteLinearOrder -.-> LinearOrder;
```
This change introduces two new auxiliary typeclasses, to encapsulate these troublesome edges. `LinearOrderedLattice` can be thought of as `LinearOrder`, but with `sup`/`inf` instead of `min`/`max`. This is crucial, because it ensures the duplicate fields are merged in `extends CompleteLattice X, LinearOrderedLattice X`, which would not be the case for `extends CompleteLattice X, LinearOrder X`. The result is:
```mermaid
graph TD
LinearOrder --> Min,Max;
LinearOrder --> LinearOrderBase;
LinearOrderBase --> PartialOrder;
Lattice --> PartialOrder;
LinearOrderedLattice -.-> LinearOrder;
LinearOrderedLattice --> LinearOrderBase;
LinearOrderedLattice --> Lattice;
CompleteLinearOrder --> LinearOrderedLattice;
ConditionallyCompleteLinearOrder --> LinearOrderedLattice;
```
---
- [ ] depends on: #23515
- [ ]
[](https://gitpod.io/from-referrer/)
|
merge-conflict |
85/66 |
Mathlib/Algebra/Order/Group/Defs.lean,Mathlib/Algebra/Order/Monoid/Defs.lean,Mathlib/Order/Basic.lean,Mathlib/Order/CompleteLattice/Defs.lean,Mathlib/Order/ConditionallyCompleteLattice/Defs.lean,Mathlib/Order/Defs/LinearOrder.lean,Mathlib/Order/Lattice.lean |
7 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
164-39114 5 months ago |
164-39114 5 months ago |
0-3019 50 minutes |
19907 |
kim-em author:kim-em |
chore: remove some 'nonrec' |
`nonrec` is nearly always obfuscatory: it tells the reader "this apparent recursive call is not actually, but I'm going to leave you to guess what it is instead", when we could just disambiguate and tell the reader.
However I'm not sure I have the patience to go through the remaining 600 uses. (A few are genuinely useful, but I guess less than 10%.) |
t-algebra
merge-conflict
label:t-algebra$ |
38/38 |
Mathlib/Algebra/Category/ModuleCat/Differentials/Basic.lean,Mathlib/Algebra/Category/ModuleCat/Differentials/Presheaf.lean,Mathlib/Algebra/CharP/ExpChar.lean,Mathlib/Algebra/ContinuedFractions/Computation/Approximations.lean,Mathlib/Algebra/ContinuedFractions/ConvergentsEquiv.lean,Mathlib/Algebra/DualNumber.lean,Mathlib/Algebra/Quaternion.lean |
7 |
2 |
['github-actions', 'kim-em'] |
nobody |
163-85887 5 months ago |
163-85887 5 months ago |
50-75559 50 days |
20746 |
JLimperg author:JLimperg |
Aesop forward branch test |
---
This is not a real PR; I just want to benchmark this Aesop branch.
[](https://gitpod.io/from-referrer/)
|
merge-conflict |
14/6 |
.github/workflows/build.yml,Mathlib/Data/Nat/Prime/Defs.lean,lake-manifest.json,lakefile.lean,scripts/bench/fake-root/lib/lean/libleanshared.so,scripts/bench/run |
6 |
11 |
['JLimperg', 'Kha', 'github-actions', 'leanprover-bot'] |
nobody |
163-82920 5 months ago |
221-65873 7 months ago |
0-0 0 seconds |
22810 |
pechersky author:pechersky |
feat(Counterexamples): metric space not induced by norm |
Because the distance is not homogeneous
---
[](https://gitpod.io/from-referrer/)
- [x] depends on: #22845 |
t-analysis
t-topology
merge-conflict
WIP
|
202/1 |
Counterexamples.lean,Counterexamples/NotBoundedSMulMetricSpace.lean,Mathlib.lean,Mathlib/Analysis/Normed/PiNat.lean,Mathlib/Topology/Algebra/Module/LocallyConvex.lean,Mathlib/Topology/MetricSpace/Polish.lean |
6 |
21 |
['eric-wieser', 'github-actions', 'loefflerd', 'mathlib4-dependent-issues-bot', 'pechersky'] |
nobody |
163-75576 5 months ago |
163-75604 5 months ago |
0-84180 23 hours |
13124 |
FR-vdash-bot author:FR-vdash-bot |
chore: remove `CovariantClass` and `ContravariantClass` |
Lean cannot handle `CovariantClass` and `ContravariantClass` correctly
- TC slowness
- [Zulip](https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/TC.20slowness)
- https://github.com/leanprover-community/mathlib4/issues/6646#issuecomment-1691792488
- It may also have made #6326 fail.
- Needs a weird hack to find instance: #9252
---
- [x] depends on: #13154
[](https://gitpod.io/from-referrer/)
|
merge-conflict
WIP
|
602/486 |
Mathlib/Algebra/AddConstMap/Basic.lean,Mathlib/Algebra/Algebra/Operations.lean,Mathlib/Algebra/Algebra/Subalgebra/Pointwise.lean,Mathlib/Algebra/BigOperators/Group/Finset/Basic.lean,Mathlib/Algebra/BigOperators/Group/Multiset/Basic.lean,Mathlib/Algebra/Group/Subgroup/Pointwise.lean,Mathlib/Algebra/Group/Submonoid/Pointwise.lean,Mathlib/Algebra/Group/UniqueProds/Basic.lean,Mathlib/Algebra/Module/Submodule/Pointwise.lean,Mathlib/Algebra/MonoidAlgebra/Degree.lean,Mathlib/Algebra/Order/AddTorsor.lean,Mathlib/Algebra/Order/Group/Action.lean,Mathlib/Algebra/Order/Group/DenselyOrdered.lean,Mathlib/Algebra/Order/Group/Units.lean,Mathlib/Algebra/Order/GroupWithZero/Canonical.lean,Mathlib/Algebra/Order/GroupWithZero/Unbundled.lean,Mathlib/Algebra/Order/GroupWithZero/WithZero.lean,Mathlib/Algebra/Order/Monoid/Defs.lean,Mathlib/Algebra/Order/Monoid/Unbundled/Basic.lean,Mathlib/Algebra/Order/Monoid/Unbundled/Defs.lean,Mathlib/Algebra/Order/Monoid/Unbundled/OrderDual.lean,Mathlib/Algebra/Order/Monoid/Unbundled/WithTop.lean,Mathlib/Algebra/Order/Ring/Defs.lean,Mathlib/Algebra/Order/Ring/WithTop.lean,Mathlib/Algebra/Ring/Subring/Pointwise.lean,Mathlib/Algebra/Ring/Subsemiring/Pointwise.lean,Mathlib/Analysis/SumOverResidueClass.lean,Mathlib/Data/DFinsupp/Lex.lean,Mathlib/Data/Finsupp/Lex.lean,Mathlib/Data/NNRat/Defs.lean,Mathlib/GroupTheory/OrderOfElement.lean,Mathlib/Order/Filter/IsBounded.lean,Mathlib/Order/Filter/Pointwise.lean,Mathlib/Probability/Kernel/Defs.lean,Mathlib/RingTheory/Ideal/Pointwise.lean,Mathlib/RingTheory/Valuation/ValuationSubring.lean,Mathlib/Topology/Algebra/Order/LiminfLimsup.lean |
37 |
6 |
['FR-vdash-bot', 'MichaelStollBayreuth', 'github-actions', 'leanprover-bot', 'mathlib4-dependent-issues-bot'] |
nobody |
163-17153 5 months ago |
163-17153 5 months ago |
0-1769 29 minutes |
20401 |
RemyDegenne author:RemyDegenne |
feat: add sigmaFinite_iUnion |
```lean
lemma sigmaFinite_iUnion (μ : Measure α) {s : ℕ → Set α} (h_meas : MeasurableSet (⋃ n, s n))
[∀ n, SigmaFinite (μ.restrict (s n))] :
SigmaFinite (μ.restrict (⋃ n, s n))
```
---
[](https://gitpod.io/from-referrer/)
|
t-measure-probability
merge-conflict
awaiting-author
|
37/28 |
Mathlib/MeasureTheory/Decomposition/Exhaustion.lean,Mathlib/MeasureTheory/Measure/Typeclasses.lean |
2 |
4 |
['RemyDegenne', 'github-actions', 'sgouezel'] |
nobody |
162-22307 5 months ago |
162-22308 5 months ago |
0-73190 20 hours |
19275 |
eric-wieser author:eric-wieser |
fix: if nolint files change, do a full rebuild |
Otherwise CI will succeed when removing entries from the file, but fail later when someone changes something unrelated.
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict
delegated
|
8/0 |
lakefile.lean |
1 |
20 |
['YaelDillies', 'adomani', 'eric-wieser', 'github-actions', 'grunweg', 'mathlib-bors'] |
nobody |
161-72875 5 months ago |
161-72875 5 months ago |
0-214 3 minutes |
12251 |
ScottCarnahan author:ScottCarnahan |
refactor(RingTheory/HahnSeries) : several generalizations |
This PR is a container for several smaller PRs that refactor and generalize the existing Hahn series theory. It is (I think) all we need from Hahn series to get a palatable theory of vertex algebras off the ground (other prerequisites from Lie algebras will eventually come in a different PR). Major changes include:
- equivalence between iterated Hahn series and Hahn series on Lex products.
- introduce `orderTop` and `leadingCoeff` functions. Here, `orderTop` is a `WithTop Γ`-valued version of `order` that does not need `[Zero Γ]` and `leadingCoeff` returns the coefficient of the minimal element of support (or zero if empty).
- introduce ordered and cancellative vector addition classes together with some basic theory e.g., finiteness of antidiagonals for partially well-ordered sets.
- `HahnSeries Γ R`-module structure on `HahnModule Γ' R V`, when `Γ` is an `OrderedCancelAddCommMonoid`, `Γ'` is a `PartialOrder` with `OrderedCancelVAdd Γ Γ'`, `R` is a semiring, and `V` is an `R`-module.
- Move `AddVal` to a separate file - the underlying function is just `orderTop`, but the description of the valuation needs an additional import and an `IsDomain` hypothesis. Results that depended on `AddVal` are changed to use `orderTop` and generalized.
---
- [x] depends on: #10781 [HahnSeries on Lex product]
- [x] depends on: #10846 [HahnModule]
- [x] depends on: #11965 [orderTop]
- [x] depends on: #11979 [OrderedVAdd]
- [x] depends on: #12996 [leadingTerm]
- [x] depends on: #16649
- [x] depends on: #16701
- [x] depends on: #17004
[](https://gitpod.io/from-referrer/)
|
t-order
t-algebra
merge-conflict
WIP
label:t-algebra$ |
1059/97 |
Mathlib/RingTheory/HahnSeries/Addition.lean,Mathlib/RingTheory/HahnSeries/Basic.lean,Mathlib/RingTheory/HahnSeries/HEval.lean,Mathlib/RingTheory/HahnSeries/Multiplication.lean,Mathlib/RingTheory/HahnSeries/PowerSeries.lean,Mathlib/RingTheory/HahnSeries/Summable.lean |
6 |
n/a |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
161-59296 5 months ago |
unknown |
unknown |
22727 |
grunweg author:grunweg |
feat: rewrite the isolated by and colon linters in Lean |
---
- depends on #22726
- depends on: #22728
[](https://gitpod.io/from-referrer/)
|
t-linter
merge-conflict
awaiting-author
|
128/96 |
Mathlib/AlgebraicTopology/SimplexCategory/GeneratorsRelations/Basic.lean,Mathlib/Data/Finsupp/AList.lean,Mathlib/Data/Int/ModEq.lean,Mathlib/Data/List/Nodup.lean,Mathlib/Data/List/TFAE.lean,Mathlib/Data/Matroid/Circuit.lean,Mathlib/Data/Matroid/Minor/Basic.lean,Mathlib/GroupTheory/Perm/Cycle/Factors.lean,Mathlib/LinearAlgebra/TensorProduct/Vanishing.lean,Mathlib/Order/KrullDimension.lean,Mathlib/Probability/Kernel/WithDensity.lean,Mathlib/RingTheory/NoetherNormalization.lean,Mathlib/Tactic/Linter/TextBased.lean,Mathlib/Topology/Sets/OpenCover.lean,scripts/lint-style.py |
15 |
3 |
['adomani', 'github-actions', 'grunweg'] |
nobody |
160-48593 5 months ago |
160-48593 5 months ago |
10-50342 10 days |
22027 |
vihdzp author:vihdzp |
chore(SetTheory/Ordinal/FixedPoint); review `Ordinal.nfp` API |
This PR does the following:
- add `iff` variants of various theorems, renaming some in the process
- weaken some assumptions slightly
- golf throughout
---
- [x] depends on: #22017
[](https://gitpod.io/from-referrer/)
|
t-set-theory
merge-conflict
|
64/61 |
Mathlib/Logic/Equiv/List.lean,Mathlib/SetTheory/Ordinal/FixedPoint.lean |
2 |
3 |
['github-actions', 'grunweg', 'mathlib4-dependent-issues-bot'] |
nobody |
160-48466 5 months ago |
163-15426 5 months ago |
43-68322 43 days |
15212 |
victorliu5296 author:victorliu5296 |
feat: Add fundamental theorem of calculus-2 for Banach spaces |
add the Mean Value Theorem for Banach spaces to the library and include reference for the theorem statement
This theorem states that if `f : X → Y` is differentiable along the line segment from `a` to `b`, then the change in `f` equals the integral of its derivative along this path. This extends the mean value theorem to Banach spaces. This can be used for the eventual proof of the Newton-Kantorovich theorem with 1 constant contained inside the added reference.
Here is the discussion on Zulipchat: https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/Contributing.20FTC-2.20for.20Banach.20spaces |
new-contributor
t-measure-probability
t-analysis
merge-conflict
awaiting-author
|
60/1 |
Mathlib/MeasureTheory/Integral/FundThmCalculus.lean |
1 |
3 |
['github-actions', 'hrmacbeth', 'victorliu5296'] |
nobody |
160-8273 5 months ago |
160-8273 5 months ago |
51-85104 51 days |
22701 |
ctchou author:ctchou |
feat(Combinatorics): the Katona circle method |
This file formalizes the Katona circle method.
From PlainCombi (LeanCamCombi): https://github.com/YaelDillies/LeanCamCombi/blob/master/LeanCamCombi/PlainCombi/KatonaCircle.lean
Co-authored-by: Yaël Dillies
|
new-contributor
t-combinatorics
merge-conflict
|
121/0 |
Mathlib.lean,Mathlib/Combinatorics/KatonaCircle.lean |
2 |
1 |
['github-actions'] |
nobody |
159-44228 5 months ago |
159-44228 5 months ago |
30-8337 30 days |
23402 |
mattrobball author:mattrobball |
refactor(LinearAlgebra.TensorProduct): make `TensorProduct` irreducible |
Mathematicians generally do not reason about tensor products using a particular model, precisely because the universal properties are more natural and the precise instantiations are too complicated for most purposes. Similarly, we shouldn't allow Lean to look inside `TensorProduct` and encourage building API on top of it to avoid definitional abuse.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
label:t-algebra$ |
124/69 |
Mathlib/Algebra/Category/ModuleCat/ChangeOfRings.lean,Mathlib/Algebra/Category/ModuleCat/Monoidal/Basic.lean,Mathlib/Algebra/Category/Ring/Constructions.lean,Mathlib/LinearAlgebra/Alternating/DomCoprod.lean,Mathlib/LinearAlgebra/QuadraticForm/TensorProduct.lean,Mathlib/LinearAlgebra/QuadraticForm/TensorProduct/Isometries.lean,Mathlib/LinearAlgebra/TensorProduct/Basic.lean,Mathlib/LinearAlgebra/TensorProduct/Subalgebra.lean,Mathlib/LinearAlgebra/TensorProduct/Tower.lean,Mathlib/RingTheory/Bialgebra/TensorProduct.lean,Mathlib/RingTheory/Coalgebra/TensorProduct.lean,Mathlib/RingTheory/Kaehler/CotangentComplex.lean,Mathlib/RingTheory/Kaehler/JacobiZariski.lean,Mathlib/RingTheory/LocalRing/Module.lean,Mathlib/RingTheory/TensorProduct/Basic.lean |
15 |
8 |
['eric-wieser', 'github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'mattrobball'] |
nobody |
159-12533 5 months ago |
159-12534 5 months ago |
0-0 0 seconds |
15943 |
urkud author:urkud |
feat: add `ProdQuotientMapSpace` |
---
[](https://gitpod.io/from-referrer/)
|
t-topology
merge-conflict
|
731/11 |
Mathlib.lean,Mathlib/Topology/Basic.lean,Mathlib/Topology/Compactness/Compact.lean,Mathlib/Topology/Maps/ProdQuotient.lean |
4 |
2 |
['github-actions', 'leanprover-community-bot-assistant'] |
nobody |
158-26645 5 months ago |
158-26648 5 months ago |
0-0 0 seconds |
23786 |
grunweg author:grunweg |
Mr librarynote def 2b |
---
[](https://gitpod.io/from-referrer/)
|
large-import
merge-conflict
WIP
|
510/484 |
Archive/Imo/Imo2019Q2.lean,Mathlib/Algebra/Algebra/Basic.lean,Mathlib/Algebra/Algebra/Defs.lean,Mathlib/Algebra/Algebra/Equiv.lean,Mathlib/Algebra/Algebra/Hom.lean,Mathlib/Algebra/Algebra/NonUnitalHom.lean,Mathlib/Algebra/Algebra/NonUnitalSubalgebra.lean,Mathlib/Algebra/Algebra/ZMod.lean,Mathlib/Algebra/BigOperators/Group/Finset/Defs.lean,Mathlib/Algebra/Category/Ring/Limits.lean,Mathlib/Algebra/Colimit/Ring.lean,Mathlib/Algebra/EuclideanDomain/Basic.lean,Mathlib/Algebra/Field/MinimalAxioms.lean,Mathlib/Algebra/Field/Subfield/Defs.lean,Mathlib/Algebra/Group/Action/Defs.lean,Mathlib/Algebra/Group/Action/End.lean,Mathlib/Algebra/Group/Action/Hom.lean,Mathlib/Algebra/Group/Conj.lean,Mathlib/Algebra/Group/Defs.lean,Mathlib/Algebra/Group/Equiv/Defs.lean,Mathlib/Algebra/Group/Hom/Defs.lean,Mathlib/Algebra/Group/InjSurj.lean,Mathlib/Algebra/Group/MinimalAxioms.lean,Mathlib/Algebra/Group/Pointwise/Set/Basic.lean,Mathlib/Algebra/Group/Pointwise/Set/Scalar.lean,Mathlib/Algebra/Group/Submonoid/Operations.lean,Mathlib/Algebra/Group/Units/Defs.lean,Mathlib/Algebra/Group/Units/Hom.lean,Mathlib/Algebra/GroupWithZero/Action/Defs.lean,Mathlib/Algebra/GroupWithZero/Action/End.lean,Mathlib/Algebra/GroupWithZero/Basic.lean,Mathlib/Algebra/GroupWithZero/Defs.lean,Mathlib/Algebra/GroupWithZero/Equiv.lean,Mathlib/Algebra/GroupWithZero/InjSurj.lean,Mathlib/Algebra/GroupWithZero/Units/Basic.lean,Mathlib/Algebra/HierarchyDesign.lean,Mathlib/Algebra/Lie/Basic.lean,Mathlib/Algebra/Lie/Derivation/Basic.lean,Mathlib/Algebra/Lie/OfAssociative.lean,Mathlib/Algebra/Module/Defs.lean,Mathlib/Algebra/Module/Equiv/Defs.lean,Mathlib/Algebra/Module/NatInt.lean,Mathlib/Algebra/Module/Rat.lean,Mathlib/Algebra/Module/RingHom.lean,Mathlib/Algebra/Module/ZMod.lean,Mathlib/Algebra/NoZeroSMulDivisors/Basic.lean,Mathlib/Algebra/NoZeroSMulDivisors/Defs.lean,Mathlib/Algebra/Order/Field/Defs.lean,Mathlib/Algebra/Order/Group/Defs.lean,Mathlib/Algebra/Order/Group/InjSurj.lean,Mathlib/Algebra/Order/GroupWithZero/Canonical.lean,Mathlib/Algebra/Order/Hom/Basic.lean,Mathlib/Algebra/Order/Hom/Ring.lean,Mathlib/Algebra/Order/Kleene.lean,Mathlib/Algebra/Order/Module/Defs.lean,Mathlib/Algebra/Order/Monoid/Basic.lean,Mathlib/Algebra/Order/Monoid/Defs.lean,Mathlib/Algebra/Order/Monoid/Unbundled/ExistsOfLE.lean,Mathlib/Algebra/Order/Ring/Defs.lean,Mathlib/Algebra/Order/Ring/Star.lean,Mathlib/Algebra/Order/Star/Basic.lean,Mathlib/Algebra/Order/Sub/Basic.lean,Mathlib/Algebra/Ring/Action/Basic.lean,Mathlib/Algebra/Ring/Equiv.lean,Mathlib/Algebra/Ring/InjSurj.lean,Mathlib/Algebra/Ring/MinimalAxioms.lean,Mathlib/Algebra/Ring/Subring/Defs.lean,Mathlib/Algebra/Ring/Subsemiring/Defs.lean,Mathlib/Algebra/Star/NonUnitalSubalgebra.lean,Mathlib/Algebra/Star/StarAlgHom.lean,Mathlib/Algebra/Star/StarRingHom.lean,Mathlib/Algebra/Star/Subalgebra.lean,Mathlib/AlgebraicGeometry/Scheme.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Note.lean,Mathlib/Analysis/CStarAlgebra/Spectrum.lean,Mathlib/Analysis/Convex/Uniform.lean,Mathlib/Analysis/InnerProductSpace/Convex.lean,Mathlib/Analysis/InnerProductSpace/OfNorm.lean,Mathlib/Analysis/InnerProductSpace/Projection.lean,Mathlib/Analysis/Normed/Field/Basic.lean,Mathlib/Analysis/Normed/Group/Basic.lean,Mathlib/Analysis/Normed/Group/Constructions.lean,Mathlib/Analysis/Normed/Group/Seminorm.lean,Mathlib/Analysis/Normed/Group/Uniform.lean,Mathlib/Analysis/Normed/Lp/PiLp.lean,Mathlib/Analysis/Normed/Lp/ProdLp.lean,Mathlib/Analysis/Normed/Module/Basic.lean,Mathlib/Analysis/Normed/Operator/LinearIsometry.lean,Mathlib/Analysis/Normed/Order/Lattice.lean,Mathlib/Analysis/Normed/Ring/Basic.lean,Mathlib/Analysis/RCLike/Lemmas.lean,Mathlib/CategoryTheory/Category/Basic.lean,Mathlib/CategoryTheory/Comma/Over/OverClass.lean,Mathlib/CategoryTheory/Monoidal/Skeleton.lean,Mathlib/CategoryTheory/MorphismProperty/Comma.lean,Mathlib/Data/Fintype/Card.lean,Mathlib/Data/FunLike/Fintype.lean,Mathlib/Data/NNRat/Defs.lean,Mathlib/Data/Nat/Cast/Defs.lean,Mathlib/Data/Nat/Init.lean |
180 |
2 |
['github-actions', 'leanprover-community-bot-assistant'] |
nobody |
158-18746 5 months ago |
158-18748 5 months ago |
0-0 0 seconds |
23411 |
PatrickMassot author:PatrickMassot |
chore: remove finiteness from Order.Filter.Lift |
Co-authored-by: Anatole Dedecker
---
[](https://gitpod.io/from-referrer/)
|
longest-pole
t-topology
merge-conflict
|
48/21 |
Mathlib/Dynamics/TopologicalEntropy/DynamicalEntourage.lean,Mathlib/Order/Filter/Basic.lean,Mathlib/Order/Filter/Finite.lean,Mathlib/Order/Filter/Lift.lean,Mathlib/Order/Filter/SmallSets.lean,Mathlib/Topology/Algebra/ContinuousMonoidHom.lean,Mathlib/Topology/Basic.lean |
7 |
4 |
['Vierkantor', 'github-actions', 'kim-em', 'leanprover-community-bot-assistant'] |
nobody |
158-4542 5 months ago |
158-24111 5 months ago |
10-21608 10 days |
22579 |
kvanvels author:kvanvels |
doc(Topology/Defs/Induced): fix comments on three functions related to RestrictGenTopology |
---
[](https://gitpod.io/from-referrer/)
|
t-topology
merge-conflict
awaiting-author
documentation
|
10/9 |
Mathlib/Topology/Defs/Induced.lean,Mathlib/Topology/RestrictGen.lean |
2 |
4 |
['github-actions', 'kvanvels', 'leanprover-community-bot-assistant', 'urkud'] |
nobody |
157-15176 5 months ago |
157-15178 5 months ago |
12-18679 12 days |
19771 |
robertylewis author:robertylewis |
perf: qqify two functions in linarith |
---
[](https://gitpod.io/from-referrer/)
|
t-meta
merge-conflict
|
17/24 |
Mathlib/Tactic/Linarith/Frontend.lean,Mathlib/Tactic/Linarith/Verification.lean |
2 |
5 |
['github-actions', 'grunweg', 'leanprover-bot', 'leanprover-community-bot-assistant', 'robertylewis'] |
nobody |
156-81082 5 months ago |
156-81083 5 months ago |
0-0 0 seconds |
22308 |
plp127 author:plp127 |
feat (Analysis/Convex): Generalize `Convex` lemmas to `StarConvex` |
This PR generalizes many lemmas assuming `Convex 𝕜 s` to assume `StarConvex 𝕜 0 s`.
---
- [x] depends on: #22421
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-analysis
merge-conflict
WIP
|
30/18 |
Mathlib/Analysis/Convex/Gauge.lean,Mathlib/Analysis/Convex/GaugeRescale.lean,Mathlib/Analysis/Convex/Star.lean,Mathlib/Analysis/LocallyConvex/AbsConvexOpen.lean |
4 |
5 |
['Paul-Lez', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
156-80593 5 months ago |
156-80595 5 months ago |
0-0 0 seconds |
21488 |
imbrem author:imbrem |
feat(CategoryTheory/Monoidal): premonoidal categories |
Add support for premonoidal categories
---
Still want to add support for:
- Premonoidal braided/symmetric categories
- The monoidal coherence theorem, which I've already ported in my `discretion` library
- The `coherence` tactic, which should work fine for premonoidal categories too
but wanted to get this in front of reviewers ASAP to make sure my general approach was alright
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-category-theory
merge-conflict
|
900/361 |
Mathlib/Algebra/Category/ModuleCat/Presheaf/Monoidal.lean,Mathlib/CategoryTheory/Bicategory/End.lean,Mathlib/CategoryTheory/GradedObject/Monoidal.lean,Mathlib/CategoryTheory/Localization/Monoidal.lean,Mathlib/CategoryTheory/Monoidal/Braided/Basic.lean,Mathlib/CategoryTheory/Monoidal/Category.lean,Mathlib/CategoryTheory/Monoidal/Center.lean,Mathlib/CategoryTheory/Monoidal/CoherenceLemmas.lean,Mathlib/CategoryTheory/Monoidal/Discrete.lean,Mathlib/CategoryTheory/Monoidal/End.lean,Mathlib/CategoryTheory/Monoidal/Free/Basic.lean,Mathlib/CategoryTheory/Monoidal/Functor.lean,Mathlib/CategoryTheory/Monoidal/FunctorCategory.lean,Mathlib/CategoryTheory/Monoidal/Mon_.lean,Mathlib/CategoryTheory/Monoidal/Opposite.lean,Mathlib/CategoryTheory/Monoidal/Transport.lean,Mathlib/Tactic/CategoryTheory/Monoidal/Datatypes.lean,Mathlib/Tactic/CategoryTheory/Monoidal/Normalize.lean,Mathlib/Tactic/CategoryTheory/Monoidal/PureCoherence.lean,Mathlib/Tactic/CategoryTheory/MonoidalComp.lean,MathlibTest/StringDiagram.lean |
21 |
9 |
['YaelDillies', 'github-actions', 'grunweg', 'imbrem', 'kim-em', 'leanprover-community-bot-assistant'] |
nobody |
156-76861 5 months ago |
156-76862 5 months ago |
58-20339 58 days |
21525 |
sinhp author:sinhp |
feat(CategoryTheory): Locally Cartesian Closed Categories (Prelim) |
This PR defines the basic preliminaries for defining locally cartesian closed categories (LCCCs). In particular, using the calculus of mates we define certain natural isomorphisms involving `Over.star` and `Over.pullback` which will be crucial in defining the right adjoint to the pullback functor in the development of LCCCs.
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-category-theory
merge-conflict
|
338/24 |
Mathlib/CategoryTheory/Comma/Over/Basic.lean,Mathlib/CategoryTheory/Comma/Over/Pullback.lean,Mathlib/CategoryTheory/Galois/Examples.lean |
3 |
13 |
['b-mehta', 'github-actions', 'joelriou', 'leanprover-community-bot-assistant', 'sinhp'] |
nobody |
156-76859 5 months ago |
156-76861 5 months ago |
43-83249 43 days |
13653 |
adomani author:adomani |
feat: the unusedSetOptionIn linter |
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-linter
merge-conflict
|
199/0 |
Mathlib.lean,Mathlib/Algebra/Homology/HomotopyCategory/Triangulated.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter.lean,Mathlib/Tactic/Linter/UnnecessarySetOptionIn.lean,MathlibTest/UnnecessarySetOptionIn.lean |
6 |
15 |
['adomani', 'github-actions', 'grunweg', 'leanprover-community-bot-assistant'] |
nobody |
156-21297 5 months ago |
156-21299 5 months ago |
0-0 0 seconds |
19425 |
hrmacbeth author:hrmacbeth |
perf: gcongr forward-reasoning adjustment |
This PR changes the "forward-reasoning" component of `gcongr`, rendering it more efficient, particularly in problems with a large number of variables/hypotheses in the context.
Previously `gcongr` attempted to match *every* `LocalDecl` against *every* node in the parse tree using *each* of the five implemented `@[gcongr_forward]` mini-tactics: matching directly, matching after applying `symm`, matching after applying `le_of_lt`, etc etc.
The new algorithm filters out the non-Prop `LocalDecl`s, and also adjusts the `@[gcongr_forward]` extensions so that, rather than re-apply the relevant lemmas (`symm`, `le_of_lt`, etc) at every node in the parse tree, the lemmas are applied in advance to the `LocalDecl`s and the result (if successful) stored.
The performance effect on mathlib as a whole is miniscule, but it speeds up the profiler's count of "tactic execution of Mathlib.Tactic.GCongr" in the newly-added test from 257 ms to 47 ms, and has a similar effect on real-life examples in an analysis project of mine.
Co-authored-by: Mario Carneiro
---
[](https://gitpod.io/from-referrer/)
(Note that Mario provided the ideas but not the code, so please review with appropriate diligence!) |
merge-conflict
awaiting-author
|
130/59 |
Mathlib/Order/Lattice.lean,Mathlib/Tactic/GCongr/Core.lean,Mathlib/Tactic/GCongr/ForwardAttr.lean,MathlibTest/GCongr/inequalities.lean |
4 |
17 |
['Vierkantor', 'github-actions', 'hrmacbeth', 'leanprover-bot', 'leanprover-community-bot-assistant'] |
Vierkantor assignee:Vierkantor |
156-2993 5 months ago |
156-2995 5 months ago |
4-16654 4 days |
20873 |
vbeffara author:vbeffara |
feat(Topology/Covering): path lifting and homotopy lifting |
This proves the existence and uniqueness of path and homotopy lifts through covering maps.
---
I tried to separate as much of the proof as possible into separate PRs (which are already in Mathlib now), but the proof here relies on a monolithic construction of an explicit lift along a well-chosen subdivision, in `partial_lift`, with associated definitions. Only one standalone lean file added.
An older WIP PR #10084 by Junyan Xu @alreadydone proves similar results using a very similar construction for path lifting, with a different argument to obtain continuity for homotopy lifting.
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-topology
merge-conflict
awaiting-author
|
281/1 |
Mathlib.lean,Mathlib/Topology/Covering/Basic.lean,Mathlib/Topology/Covering/Lift.lean |
3 |
9 |
['alreadydone', 'github-actions', 'grunweg', 'vbeffara'] |
nobody |
155-79589 5 months ago |
155-79589 5 months ago |
55-53553 55 days |
22817 |
peabrainiac author:peabrainiac |
feat(CategoryTheory/Sites): local sites |
Defines local sites and shows that sheaves of types on them form a local topos, in that the global sections functor `Sheaf.Γ` has a right adjoint `Sheaf.codisc` that is fully faithful.
---
- [x] depends on: #22816
[](https://gitpod.io/from-referrer/)
|
t-category-theory
merge-conflict
WIP
|
263/0 |
Mathlib.lean,Mathlib/CategoryTheory/Limits/FunctorCategory/Shapes/Products.lean,Mathlib/CategoryTheory/Limits/Types.lean,Mathlib/CategoryTheory/Sites/GlobalSections.lean,Mathlib/CategoryTheory/Sites/LocalSite.lean,Mathlib/CategoryTheory/Sites/Sheaf.lean |
6 |
4 |
['github-actions', 'joelriou', 'mathlib4-dependent-issues-bot'] |
nobody |
155-13198 5 months ago |
155-16721 5 months ago |
0-568 9 minutes |
6252 |
michaellee94 author:michaellee94 |
feat(Geometry/Manifolds/Instances/Homeomorph): Homeomorphism maps `C^k` manifolds to `C^k` manifolds |
---
[](https://gitpod.io/from-referrer/)
|
t-differential-geometry
merge-conflict
WIP
|
116/0 |
Mathlib.lean,Mathlib/Geometry/Manifold/Instances/Graph.lean |
2 |
2 |
['leanprover-community-bot-assistant', 'michaellee94'] |
nobody |
154-74054 5 months ago |
154-74056 5 months ago |
1-44375 1 day |
23867 |
kim-em author:kim-em |
chore: remove unnecessary `[AtLeastTwo n]` hypotheses |
This PR is a follow-up to #23866, demonstrating that we can remove nearly all the `[AtLeastTwo n]` hypotheses across Mathlib. |
bench-after-CI
merge-conflict
|
272/278 |
Mathlib/Algebra/AddConstMap/Basic.lean,Mathlib/Algebra/CharP/Defs.lean,Mathlib/Algebra/CharP/Invertible.lean,Mathlib/Algebra/DirectSum/Internal.lean,Mathlib/Algebra/DirectSum/Ring.lean,Mathlib/Algebra/Group/Hom/End.lean,Mathlib/Algebra/Group/Opposite.lean,Mathlib/Algebra/Group/ULift.lean,Mathlib/Algebra/Module/LinearMap/End.lean,Mathlib/Algebra/Module/NatInt.lean,Mathlib/Algebra/MonoidAlgebra/ToDirectSum.lean,Mathlib/Algebra/Order/Floor/Ring.lean,Mathlib/Algebra/Order/Floor/Semiring.lean,Mathlib/Algebra/Order/Kleene.lean,Mathlib/Algebra/Order/Monoid/Unbundled/WithTop.lean,Mathlib/Algebra/Order/Round.lean,Mathlib/Algebra/Order/SuccPred/WithBot.lean,Mathlib/Algebra/Polynomial/Basic.lean,Mathlib/Algebra/Polynomial/Coeff.lean,Mathlib/Algebra/Polynomial/Degree/Definitions.lean,Mathlib/Algebra/Polynomial/Derivative.lean,Mathlib/Algebra/Polynomial/Eval/Defs.lean,Mathlib/Algebra/Quaternion.lean,Mathlib/Algebra/Ring/Center.lean,Mathlib/Algebra/Star/Basic.lean,Mathlib/Algebra/Star/SelfAdjoint.lean,Mathlib/AlgebraicTopology/FundamentalGroupoid/Basic.lean,Mathlib/Analysis/Complex/Basic.lean,Mathlib/Analysis/Normed/Group/Basic.lean,Mathlib/Analysis/RCLike/Basic.lean,Mathlib/Analysis/SpecialFunctions/Complex/Arg.lean,Mathlib/Analysis/SpecialFunctions/Complex/Log.lean,Mathlib/Analysis/SpecialFunctions/Gamma/Basic.lean,Mathlib/Analysis/SpecialFunctions/Pow/Complex.lean,Mathlib/Analysis/SpecialFunctions/Pow/NNReal.lean,Mathlib/Data/Complex/Basic.lean,Mathlib/Data/Complex/Norm.lean,Mathlib/Data/ENNReal/Basic.lean,Mathlib/Data/ENNReal/Real.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/Data/Int/Log.lean,Mathlib/Data/Matrix/ConjTranspose.lean,Mathlib/Data/Matrix/Diagonal.lean,Mathlib/Data/Matrix/Kronecker.lean,Mathlib/Data/Matrix/Mul.lean,Mathlib/Data/Matrix/Notation.lean,Mathlib/Data/NNRat/Defs.lean,Mathlib/Data/NNReal/Defs.lean,Mathlib/Data/Nat/Cast/Basic.lean,Mathlib/Data/Nat/Cast/Commute.lean,Mathlib/Data/Nat/Cast/Defs.lean,Mathlib/Data/Nat/Cast/Order/Basic.lean,Mathlib/Data/Nat/Cast/Order/Ring.lean,Mathlib/Data/Nat/Cast/Prod.lean,Mathlib/Data/Nat/Cast/Synonym.lean,Mathlib/Data/Nat/PartENat.lean,Mathlib/Data/Rat/Lemmas.lean,Mathlib/Data/Real/Hyperreal.lean,Mathlib/Data/Real/Irrational.lean,Mathlib/Data/ZMod/Basic.lean,Mathlib/Data/ZMod/IntUnitsPower.lean,Mathlib/Geometry/Manifold/IsManifold/Basic.lean,Mathlib/Geometry/Manifold/VectorField/Pullback.lean,Mathlib/LinearAlgebra/Dimension/Finrank.lean,Mathlib/LinearAlgebra/Matrix/PosDef.lean,Mathlib/MeasureTheory/Function/ConditionalExpectation/Basic.lean,Mathlib/NumberTheory/LucasLehmer.lean,Mathlib/NumberTheory/Padics/PadicNumbers.lean,Mathlib/NumberTheory/Zsqrtd/Basic.lean,Mathlib/Order/Filter/Germ/Basic.lean,Mathlib/RingTheory/Multiplicity.lean,Mathlib/SetTheory/Cardinal/Aleph.lean,Mathlib/SetTheory/Cardinal/Basic.lean,Mathlib/SetTheory/Cardinal/Continuum.lean,Mathlib/SetTheory/Cardinal/ENat.lean,Mathlib/SetTheory/Cardinal/Order.lean,Mathlib/SetTheory/Cardinal/ToNat.lean,Mathlib/SetTheory/Game/Birthday.lean,Mathlib/SetTheory/Game/Short.lean,Mathlib/SetTheory/Ordinal/Arithmetic.lean,Mathlib/SetTheory/Ordinal/Basic.lean,Mathlib/Tactic/ENatToNat.lean,Mathlib/Topology/Algebra/Module/LinearMap.lean,Mathlib/Topology/Algebra/SeparationQuotient/Basic.lean,Mathlib/Topology/ContinuousMap/Bounded/Normed.lean,Mathlib/Topology/Instances/ENNReal/Lemmas.lean |
86 |
2 |
['github-actions', 'leanprover-community-bot-assistant'] |
nobody |
153-20431 5 months ago |
153-20433 5 months ago |
3-60152 3 days |
16314 |
FR-vdash-bot author:FR-vdash-bot |
chore(Data/Quot): deprecate `ind*'` APIs |
---
- [x] depends on: #16264
[](https://gitpod.io/from-referrer/)
|
t-data
merge-conflict
|
247/287 |
Counterexamples/CliffordAlgebraNotInjective.lean,Mathlib/Algebra/Colimit/Module.lean,Mathlib/Algebra/Lie/Quotient.lean,Mathlib/Algebra/Module/Torsion.lean,Mathlib/Algebra/RingQuot.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Angle.lean,Mathlib/CategoryTheory/ConnectedComponents.lean,Mathlib/CategoryTheory/Subobject/Basic.lean,Mathlib/CategoryTheory/Subobject/FactorThru.lean,Mathlib/CategoryTheory/Subobject/Lattice.lean,Mathlib/Computability/Reduce.lean,Mathlib/Computability/Tape.lean,Mathlib/Data/List/Cycle.lean,Mathlib/Data/Multiset/MapFold.lean,Mathlib/Data/Multiset/ZeroCons.lean,Mathlib/Data/Quot.lean,Mathlib/Data/Setoid/Basic.lean,Mathlib/Data/Setoid/Partition.lean,Mathlib/FieldTheory/Fixed.lean,Mathlib/GroupTheory/Complement.lean,Mathlib/GroupTheory/Congruence/Basic.lean,Mathlib/GroupTheory/Congruence/Defs.lean,Mathlib/GroupTheory/Congruence/Hom.lean,Mathlib/GroupTheory/Coset/Basic.lean,Mathlib/GroupTheory/Coset/Defs.lean,Mathlib/GroupTheory/FreeAbelianGroup.lean,Mathlib/GroupTheory/GroupAction/Basic.lean,Mathlib/GroupTheory/GroupAction/Defs.lean,Mathlib/GroupTheory/GroupAction/Quotient.lean,Mathlib/GroupTheory/Index.lean,Mathlib/GroupTheory/MonoidLocalization/Basic.lean,Mathlib/GroupTheory/PGroup.lean,Mathlib/GroupTheory/Perm/Cycle/Concrete.lean,Mathlib/GroupTheory/PresentedGroup.lean,Mathlib/GroupTheory/QuotientGroup/Basic.lean,Mathlib/GroupTheory/QuotientGroup/Defs.lean,Mathlib/GroupTheory/SchurZassenhaus.lean,Mathlib/GroupTheory/Sylow.lean,Mathlib/LinearAlgebra/Alternating/DomCoprod.lean,Mathlib/LinearAlgebra/Projectivization/Basic.lean,Mathlib/LinearAlgebra/Quotient/Basic.lean,Mathlib/LinearAlgebra/Quotient/Defs.lean,Mathlib/MeasureTheory/Function/AEEqFun.lean,Mathlib/NumberTheory/Padics/PadicNumbers.lean,Mathlib/NumberTheory/RamificationInertia/Basic.lean,Mathlib/Order/Antisymmetrization.lean,Mathlib/Order/Category/PartOrd.lean,Mathlib/Order/Filter/Germ/Basic.lean,Mathlib/RepresentationTheory/GroupCohomology/Hilbert90.lean,Mathlib/RingTheory/AdicCompletion/Algebra.lean,Mathlib/RingTheory/AdicCompletion/Basic.lean,Mathlib/RingTheory/AdicCompletion/Functoriality.lean,Mathlib/RingTheory/AdjoinRoot.lean,Mathlib/RingTheory/Congruence/Basic.lean,Mathlib/RingTheory/Flat/FaithfullyFlat/Basic.lean,Mathlib/RingTheory/GradedAlgebra/HomogeneousLocalization.lean,Mathlib/RingTheory/Ideal/Cotangent.lean,Mathlib/RingTheory/Ideal/Norm/AbsNorm.lean,Mathlib/RingTheory/Ideal/Quotient/Basic.lean,Mathlib/RingTheory/Ideal/Quotient/Defs.lean,Mathlib/RingTheory/Ideal/Quotient/Operations.lean,Mathlib/RingTheory/Valuation/Quotient.lean,Mathlib/Topology/Algebra/Group/TopologicalAbelianization.lean,Mathlib/Topology/Algebra/InfiniteSum/Module.lean,Mathlib/Topology/Separation/Basic.lean |
65 |
4 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
151-15425 4 months ago |
151-15427 4 months ago |
55-52030 55 days |
23509 |
eric-wieser author:eric-wieser |
refactor: Make ENNReal an abbrev |
The `Coe` instance becomes `CoeTC` to match what we do for `WithTop` (such that the priority kicks in)
Probably we could have both copies and things would be ok.
---
[](https://gitpod.io/from-referrer/)
This includes part of #23750
|
t-data
merge-conflict
|
22/66 |
Mathlib/Data/ENNReal/Basic.lean,Mathlib/Data/ENNReal/BigOperators.lean,Mathlib/Data/ENNReal/Operations.lean,Mathlib/MeasureTheory/Integral/SetToL1.lean,Mathlib/MeasureTheory/Measure/Sub.lean,Mathlib/MeasureTheory/Measure/TightNormed.lean,Mathlib/Topology/MetricSpace/PartitionOfUnity.lean |
7 |
22 |
['eric-wieser', 'github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'leanprover-community-mathlib4-bot', 'mattrobball', 'urkud'] |
nobody |
150-85478 4 months ago |
150-85480 4 months ago |
14-12910 14 days |
24060 |
eric-wieser author:eric-wieser |
chore(MeasureTheory): use `0` instead of `const _ 0` |
---
[](https://gitpod.io/from-referrer/)
|
t-measure-probability
merge-conflict
|
30/20 |
Mathlib/MeasureTheory/Function/SimpleFunc.lean,Mathlib/MeasureTheory/Function/SimpleFuncDense.lean,Mathlib/MeasureTheory/Function/SimpleFuncDenseLp.lean,Mathlib/MeasureTheory/Integral/Bochner/VitaliCaratheodory.lean,Mathlib/MeasureTheory/Integral/Lebesgue/Countable.lean,Mathlib/MeasureTheory/Integral/SetToL1.lean,Mathlib/Probability/StrongLaw.lean |
7 |
2 |
['github-actions', 'leanprover-community-bot-assistant'] |
nobody |
150-75173 4 months ago |
150-75175 4 months ago |
0-0 0 seconds |
11455 |
adomani author:adomani |
fix: unsqueeze simp, re Yaël's comments on #11259 |
This PR reverts/simplifies some of the "squeeze `simp`" changes in #11259.
See #11259 for context.
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict
awaiting-author
|
3/6 |
Mathlib/Algebra/Group/Conj.lean,Mathlib/Data/Seq/WSeq.lean |
2 |
8 |
['Ruben-VandeVelde', 'YaelDillies', 'grunweg', 'loefflerd', 'robertylewis', 'urkud'] |
nobody |
150-47078 4 months ago |
420-73668 1 year ago |
91-14162 91 days |
7325 |
eric-wieser author:eric-wieser |
chore: use preimageIso instead of defeq abuse for InducedCategory |
This makes a few things slightly more verbose, but the type casts are now explicit in those places.
---
[](https://gitpod.io/from-referrer/)
|
t-category-theory
awaiting-CI
merge-conflict
|
22/21 |
Mathlib/CategoryTheory/EssentialImage.lean,Mathlib/CategoryTheory/Monoidal/Braided.lean,Mathlib/CategoryTheory/Monoidal/Subcategory.lean |
3 |
1 |
['grunweg'] |
nobody |
150-46957 4 months ago |
430-76042 1 year ago |
0-0 0 seconds |
7874 |
astrainfinita author:astrainfinita |
chore: make `IsScalarTower A A B` and `IsScalarTower A B B` higher priority |
---
[](https://gitpod.io/from-referrer/)
|
slow-typeclass-synthesis
t-algebra
awaiting-CI
merge-conflict
label:t-algebra$ |
10/9 |
Mathlib/Algebra/Algebra/Defs.lean,Mathlib/Algebra/Group/Action/Defs.lean,Mathlib/Data/Rat/Cast/Defs.lean,Mathlib/GroupTheory/GroupAction/Ring.lean |
4 |
3 |
['astrainfinita', 'grunweg', 'leanprover-bot'] |
nobody |
150-46932 4 months ago |
420-73927 1 year ago |
0-0 0 seconds |
5952 |
eric-wieser author:eric-wieser |
feat: add Qq wrappers for ToExpr |
---
- [ ] depends on: #6699 (to appease the linter)
[](https://gitpod.io/from-referrer/)
|
awaiting-CI
t-meta
merge-conflict
|
247/150 |
Mathlib/Data/Fin/Basic.lean,Mathlib/Data/Fin/VecNotation.lean,Mathlib/Data/Matrix/Notation.lean,Mathlib/Tactic/DeriveToExpr.lean,Mathlib/Tactic/FBinop.lean,Mathlib/Tactic/ToExpr.lean,Mathlib/Util/Qq.lean,test/DeriveToExpr.lean,test/vec_notation.lean |
9 |
7 |
['eric-wieser', 'gebner', 'grunweg', 'leanprover-community-mathlib4-bot'] |
nobody |
150-46758 4 months ago |
430-76042 1 year ago |
29-67421 29 days |
15483 |
FR-vdash-bot author:FR-vdash-bot |
chore(GroupTheory/Coset): reduce defeq abuse |
---
- [x] depends on: #15482
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
label:t-algebra$ |
114/60 |
Mathlib/GroupTheory/Commensurable.lean,Mathlib/GroupTheory/Coset.lean,Mathlib/GroupTheory/QuotientGroup.lean,Mathlib/LinearAlgebra/Alternating/DomCoprod.lean,Mathlib/MeasureTheory/Measure/Haar/Quotient.lean,Mathlib/Topology/Algebra/Group/Compact.lean |
6 |
14 |
['FR-vdash-bot', 'eric-wieser', 'github-actions', 'grunweg', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'mattrobball', 'mergify', 'urkud'] |
nobody |
150-46718 4 months ago |
398-85048 1 year ago |
4-79214 4 days |
16594 |
FR-vdash-bot author:FR-vdash-bot |
perf: reorder `extends` and remove some instances in algebra hierarchy |
---
[](https://gitpod.io/from-referrer/)
|
slow-typeclass-synthesis
t-algebra
merge-conflict
label:t-algebra$ |
240/92 |
Mathlib.lean,Mathlib/Algebra/Algebra/Hom.lean,Mathlib/Algebra/Associated/Basic.lean,Mathlib/Algebra/BigOperators/Ring/List.lean,Mathlib/Algebra/Field/Defs.lean,Mathlib/Algebra/GCDMonoid/Basic.lean,Mathlib/Algebra/Group/Defs.lean,Mathlib/Algebra/Group/Ext.lean,Mathlib/Algebra/Group/Opposite.lean,Mathlib/Algebra/Group/Prod.lean,Mathlib/Algebra/GroupWithZero/Defs.lean,Mathlib/Algebra/GroupWithZero/Prod.lean,Mathlib/Algebra/Homology/Embedding/Basic.lean,Mathlib/Algebra/Order/AddGroupWithTop.lean,Mathlib/Algebra/Order/Field/Canonical/Defs.lean,Mathlib/Algebra/Order/Field/Defs.lean,Mathlib/Algebra/Order/Group/Unbundled/Abs.lean,Mathlib/Algebra/Order/GroupWithZero/Canonical.lean,Mathlib/Algebra/Order/Ring/Canonical.lean,Mathlib/Algebra/Order/Ring/Defs.lean,Mathlib/Algebra/Polynomial/Roots.lean,Mathlib/Algebra/Quaternion.lean,Mathlib/Algebra/Ring/Defs.lean,Mathlib/Algebra/Ring/Ext.lean,Mathlib/Algebra/Ring/InjSurj.lean,Mathlib/Algebra/Ring/Rat.lean,Mathlib/Algebra/Ring/SumsOfSquares.lean,Mathlib/Algebra/Tropical/Basic.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Order.lean,Mathlib/Analysis/InnerProductSpace/Symmetric.lean,Mathlib/CategoryTheory/Preadditive/FunctorCategory.lean,Mathlib/Data/Finset/NoncommProd.lean,Mathlib/Data/Int/Cast/Defs.lean,Mathlib/FieldTheory/IsAlgClosed/AlgebraicClosure.lean,Mathlib/FieldTheory/SplittingField/Construction.lean,Mathlib/GroupTheory/Congruence/Basic.lean,Mathlib/GroupTheory/MonoidLocalization/MonoidWithZero.lean,Mathlib/GroupTheory/Torsion.lean,Mathlib/LinearAlgebra/LinearPMap.lean,Mathlib/LinearAlgebra/TensorProduct/Basic.lean,Mathlib/Order/Filter/Germ/Basic.lean,Mathlib/Order/Interval/Finset/Box.lean,Mathlib/RingTheory/Bialgebra/Hom.lean,Mathlib/RingTheory/Coalgebra/Hom.lean,Mathlib/RingTheory/Ideal/Quotient.lean,Mathlib/RingTheory/Perfection.lean,Mathlib/RingTheory/TensorProduct/Basic.lean,Mathlib/RingTheory/TensorProduct/MvPolynomial.lean,Mathlib/Util/NoInstances.lean,scripts/noshake.json |
50 |
8 |
['FR-vdash-bot', 'github-actions', 'grunweg', 'leanprover-bot'] |
nobody |
150-46494 4 months ago |
354-86041 11 months ago |
14-58900 14 days |
13780 |
adomani author:adomani |
deprecate injective |
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict |
31/9 |
.github/workflows/bors.yml,.github/workflows/build.yml,.github/workflows/build.yml.in,.github/workflows/build_fork.yml,Mathlib/Init/Function.lean,lake-manifest.json,lakefile.lean |
7 |
2 |
['github-actions', 'grunweg'] |
nobody |
150-14008 4 months ago |
445-83752 1 year ago |
0-0 0 seconds |
11297 |
mattrobball author:mattrobball |
mrb/cover data fields |
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict |
949/657 |
Mathlib/Algebra/Algebra/Equiv.lean,Mathlib/Algebra/Algebra/Hom.lean,Mathlib/Algebra/Associated.lean,Mathlib/Algebra/Category/MonCat/Colimits.lean,Mathlib/Algebra/Category/Ring/Colimits.lean,Mathlib/Algebra/DirectSum/Ring.lean,Mathlib/Algebra/Field/Basic.lean,Mathlib/Algebra/Field/IsField.lean,Mathlib/Algebra/Free.lean,Mathlib/Algebra/FreeMonoid/Basic.lean,Mathlib/Algebra/GradedMonoid.lean,Mathlib/Algebra/Group/Aut.lean,Mathlib/Algebra/Group/Hom/Defs.lean,Mathlib/Algebra/Group/Hom/Instances.lean,Mathlib/Algebra/Group/InjSurj.lean,Mathlib/Algebra/Group/Opposite.lean,Mathlib/Algebra/Group/Pi/Lemmas.lean,Mathlib/Algebra/Group/TypeTags.lean,Mathlib/Algebra/Group/Units.lean,Mathlib/Algebra/Group/WithOne/Defs.lean,Mathlib/Algebra/GroupWithZero/Basic.lean,Mathlib/Algebra/GroupWithZero/InjSurj.lean,Mathlib/Algebra/Lie/NonUnitalNonAssocAlgebra.lean,Mathlib/Algebra/Module/Basic.lean,Mathlib/Algebra/Module/Equiv.lean,Mathlib/Algebra/Module/LocalizedModule.lean,Mathlib/Algebra/Order/Group/Cone.lean,Mathlib/Algebra/Order/Interval.lean,Mathlib/Algebra/Order/Monoid/WithTop.lean,Mathlib/Algebra/Order/Ring/WithTop.lean,Mathlib/Algebra/PEmptyInstances.lean,Mathlib/Algebra/Quandle.lean,Mathlib/Algebra/Ring/Aut.lean,Mathlib/Algebra/Ring/Defs.lean,Mathlib/Algebra/Ring/Hom/Defs.lean,Mathlib/Algebra/Ring/InjSurj.lean,Mathlib/Algebra/Ring/Opposite.lean,Mathlib/Algebra/Ring/Pi.lean,Mathlib/Algebra/Ring/ULift.lean,Mathlib/Algebra/SMulWithZero.lean,Mathlib/Algebra/Star/StarAlgHom.lean,Mathlib/Algebra/Tropical/Basic.lean,Mathlib/Analysis/Fourier/FourierTransformDeriv.lean,Mathlib/Analysis/NormedSpace/ContinuousAffineMap.lean,Mathlib/Analysis/NormedSpace/HahnBanach/Extension.lean,Mathlib/Analysis/NormedSpace/OperatorNorm/Basic.lean,Mathlib/Analysis/SpecialFunctions/PolarCoord.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Deriv.lean,Mathlib/CategoryTheory/Endomorphism.lean,Mathlib/CategoryTheory/Groupoid/VertexGroup.lean,Mathlib/CategoryTheory/Monoidal/Internal/Module.lean,Mathlib/Combinatorics/Quiver/SingleObj.lean,Mathlib/Combinatorics/Quiver/Symmetric.lean,Mathlib/Combinatorics/Young/YoungDiagram.lean,Mathlib/Control/Applicative.lean,Mathlib/Control/Basic.lean,Mathlib/Control/Functor.lean,Mathlib/Control/Monad/Cont.lean,Mathlib/Control/ULift.lean,Mathlib/Data/Erased.lean,Mathlib/Data/Int/Basic.lean,Mathlib/Data/Int/Cast/Prod.lean,Mathlib/Data/Nat/Basic.lean,Mathlib/Data/Nat/Cast/Defs.lean,Mathlib/Data/Nat/Order/Basic.lean,Mathlib/Data/Num/Lemmas.lean,Mathlib/Data/PSigma/Order.lean,Mathlib/Data/Prod/Lex.lean,Mathlib/Data/Quot.lean,Mathlib/Data/Rat/Defs.lean,Mathlib/Data/Set/Basic.lean,Mathlib/Data/Set/Semiring.lean,Mathlib/Data/Sigma/Order.lean,Mathlib/Data/Sign.lean,Mathlib/Data/Sum/Lattice.lean,Mathlib/Data/Sum/Order.lean,Mathlib/Data/TwoPointing.lean,Mathlib/Data/ZMod/Defs.lean,Mathlib/GroupTheory/FreeGroup/Basic.lean,Mathlib/GroupTheory/GroupAction/Basic.lean,Mathlib/GroupTheory/GroupAction/Defs.lean,Mathlib/GroupTheory/GroupAction/Opposite.lean,Mathlib/GroupTheory/GroupAction/Option.lean,Mathlib/GroupTheory/GroupAction/Prod.lean,Mathlib/GroupTheory/GroupAction/SubMulAction/Pointwise.lean,Mathlib/GroupTheory/GroupAction/Units.lean,Mathlib/GroupTheory/MonoidLocalization.lean,Mathlib/GroupTheory/Perm/Basic.lean,Mathlib/GroupTheory/Subgroup/Basic.lean,Mathlib/GroupTheory/Submonoid/Operations.lean,Mathlib/GroupTheory/Submonoid/Pointwise.lean,Mathlib/GroupTheory/Subsemigroup/Operations.lean,Mathlib/Init/Data/Int/Order.lean,Mathlib/Init/Data/List/Instances.lean,Mathlib/Init/Data/Nat/Lemmas.lean,Mathlib/LinearAlgebra/AffineSpace/AffineMap.lean,Mathlib/LinearAlgebra/Basis.lean,Mathlib/Logic/Nontrivial/Basic.lean,Mathlib/Logic/Unique.lean,Mathlib/MeasureTheory/Integral/Bochner.lean |
120 |
13 |
['YaelDillies', 'grunweg', 'leanprover-bot', 'mattrobball'] |
nobody |
150-13560 4 months ago |
548-44232 1 year ago |
0-0 0 seconds |
12673 |
grunweg author:grunweg |
feat: add ContDiff.lipschitzOnWith |
A C¹ function is Lipschitz on each convex compact set. From sphere-eversion.
--------
Commits can be reviewed independently.
[](https://gitpod.io/from-referrer/)
|
t-analysis
merge-conflict
awaiting-author
help-wanted
|
30/11 |
Mathlib/Analysis/Calculus/ContDiff/RCLike.lean |
1 |
6 |
['Ruben-VandeVelde', 'github-actions', 'grunweg', 'sgouezel'] |
nobody |
148-69471 4 months ago |
148-69471 4 months ago |
1-7552 1 day |
20567 |
grunweg author:grunweg |
feat(Cache): two small features |
- add an informational message to the get command (when run without arguments):
when more than 80% of all cache files present were not used in the last command,
tell the user about the `clean` command
---
- [ ] depends on #20568 (for the first feature)
- [ ] TODO: re-design this feature and the clean command: if there are N local copies of mathlib, cache should have a pointer to all of them - to avoid clearing all N-1 from inside the last local copy
[](https://gitpod.io/from-referrer/)
|
t-meta
merge-conflict
|
38/2 |
Cache/Main.lean |
1 |
11 |
['Julian', 'arthurpaulino', 'fpvandoorn', 'github-actions', 'grunweg'] |
nobody |
148-50821 4 months ago |
148-50821 4 months ago |
1-17369 1 day |
20313 |
thefundamentaltheor3m author:thefundamentaltheor3m |
feat(Data/Complex/Exponential): prove some useful results about the complex exponential. |
This PR proves two basic results about the complex exponential:
* `abs_exp_mul_I (x : ℂ) : abs (Complex.exp (I * x)) = Real.exp (-x.im)`
* `one_sub_rexp_re_le_abs_one_sub_cexp (x : ℂ) : 1 - Real.exp x.re ≤ Complex.abs (1 - Complex.exp x)`
Both results were proved as part of the sphere packing project. There's a chance they're too specific for mathlib, but I thought they were worth PRing anyway. Would it also be a good idea to tag `abs_exp_mul_I` with `simp`? Feedback/suggestions welcome.
Note: `one_sub_rexp_re_le_abs_one_sub_cexp` was proved by Bhavik Mehta @b-mehta
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-analysis
merge-conflict
|
167/141 |
Mathlib.lean,Mathlib/Analysis/Complex/Basic.lean,Mathlib/Analysis/SpecialFunctions/Log/ERealExp.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Chebyshev.lean,Mathlib/Data/Complex/Exponential/Defs.lean,Mathlib/Data/Complex/Exponential/Lemmas.lean,Mathlib/Data/Complex/ExponentialBounds.lean,Mathlib/Tactic/FunProp.lean,MathlibTest/Recall.lean,MathlibTest/positivity.lean |
10 |
12 |
['b-mehta', 'github-actions', 'kim-em', 'thefundamentaltheor3m', 'trivial1711'] |
nobody |
148-50787 4 months ago |
148-50787 4 months ago |
25-60481 25 days |
22698 |
Kiolt author:Kiolt |
feat: notation for whisker(Left/Right)Iso |
From Toric
---
[](https://gitpod.io/from-referrer/)
|
toric
t-category-theory
merge-conflict
|
175/113 |
Mathlib/Algebra/Homology/Monoidal.lean,Mathlib/CategoryTheory/Bicategory/Adjunction/Basic.lean,Mathlib/CategoryTheory/Bicategory/Basic.lean,Mathlib/CategoryTheory/Bicategory/Coherence.lean,Mathlib/CategoryTheory/Bicategory/Extension.lean,Mathlib/CategoryTheory/Bicategory/Functor/Pseudofunctor.lean,Mathlib/CategoryTheory/Bicategory/NaturalTransformation/Strong.lean,Mathlib/CategoryTheory/Bicategory/SingleObj.lean,Mathlib/CategoryTheory/Closed/Functor.lean,Mathlib/CategoryTheory/Closed/Ideal.lean,Mathlib/CategoryTheory/Enriched/FunctorCategory.lean,Mathlib/CategoryTheory/GradedObject/Monoidal.lean,Mathlib/CategoryTheory/Monoidal/Braided/Basic.lean,Mathlib/CategoryTheory/Monoidal/Braided/Reflection.lean,Mathlib/CategoryTheory/Monoidal/Category.lean,Mathlib/CategoryTheory/Monoidal/Center.lean,Mathlib/CategoryTheory/Monoidal/Free/Coherence.lean,Mathlib/CategoryTheory/Monoidal/Preadditive.lean,Mathlib/CategoryTheory/Monoidal/Transport.lean,Mathlib/Tactic/CategoryTheory/BicategoricalComp.lean,Mathlib/Tactic/CategoryTheory/Bicategory/Datatypes.lean,Mathlib/Tactic/CategoryTheory/Bicategory/Normalize.lean,Mathlib/Tactic/CategoryTheory/Bicategory/PureCoherence.lean,Mathlib/Tactic/CategoryTheory/Monoidal/Datatypes.lean,Mathlib/Tactic/CategoryTheory/Monoidal/Normalize.lean,Mathlib/Tactic/CategoryTheory/Monoidal/PureCoherence.lean,Mathlib/Tactic/CategoryTheory/MonoidalComp.lean |
27 |
21 |
['Kiolt', 'YaelDillies', 'b-mehta', 'github-actions', 'leanprover-bot'] |
nobody |
148-50616 4 months ago |
148-50616 4 months ago |
3-36238 3 days |
21714 |
mattrobball author:mattrobball |
test |
|
t-order
merge-conflict
|
13/13 |
Mathlib/Order/Hom/Lattice.lean,lean-toolchain |
2 |
4 |
['github-actions', 'leanprover-bot', 'mattrobball'] |
nobody |
148-49465 4 months ago |
148-49465 4 months ago |
0-0 0 seconds |
20730 |
kuotsanhsu author:kuotsanhsu |
feat(LinearAlgebra/Matrix/SchurTriangulation): prove Schur decomposition/triangulation |
`Matrix.schur_triangulation` shows that a matrix over an algebraically closed field is unitarily similar to an upper triangular matrix
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-algebra
merge-conflict
awaiting-author
label:t-algebra$ |
317/2 |
Mathlib.lean,Mathlib/LinearAlgebra/Matrix/Block.lean,Mathlib/LinearAlgebra/Matrix/SchurTriangulation.lean,Mathlib/Logic/Equiv/Basic.lean |
4 |
14 |
['eric-wieser', 'github-actions', 'kim-em', 'kuotsanhsu'] |
nobody |
148-46919 4 months ago |
148-46919 4 months ago |
13-60072 13 days |
19117 |
eric-wieser author:eric-wieser |
feat: derivatives of matrix operations |
These are finally possible to state after #19108.
However, a lot of bundled `ContinuousLinearMap`s are missing.
---
- [x] depends on: #19108
[](https://gitpod.io/from-referrer/)
|
t-analysis
merge-conflict
WIP
|
336/22 |
Mathlib.lean,Mathlib/Analysis/Calculus/Deriv/Matrix.lean,Mathlib/Analysis/Calculus/FDeriv/Basic.lean,Mathlib/Analysis/Calculus/FDeriv/Matrix.lean |
4 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
146-69297 4 months ago |
146-69299 4 months ago |
0-0 0 seconds |
12605 |
FR-vdash-bot author:FR-vdash-bot |
chore: attribute [induction_eliminator] |
Add attribute [induction_eliminator] to
`AdjoinRoot.induction_on`
`ENat.recTopCoe`
`ENNReal.recTopCoe`
`Finset.induction`
`Magma.AssocQuotient.induction_on`
`ManyOneDegree.ind_on`
`Module.Ray.ind` (and add `Orientation.ind` for `Orientation`, an abbrev of it. I wish that we do not need to add it in the future.)
`Multiset.induction`
`MvPolynomial.induction_on`
`OnePoint.rec`
`Opposite.rec'`
`Ordinal.limitRecOn`
`PartENat.casesOn`
`Polynomial.induction_on'`
`QuotientAddGroup.induction_on'` (and add `AddCircle.induction_on` for `AddCircle`, an abbrev of it. I wish that we do not need to add it in the future.)
`QuotientGroup.induction_on'` (doesn't actually work)
`Real.Angle.induction_on`
`SimplexCategory.rec`
`Trunc.induction_on`
---
- [x] depends on: #13476
- [x] depends on: #13264
[](https://gitpod.io/from-referrer/)
|
merge-conflict
awaiting-author
|
354/342 |
Mathlib/Algebra/BigOperators/Associated.lean,Mathlib/Algebra/BigOperators/Group/Finset.lean,Mathlib/Algebra/BigOperators/Group/Multiset.lean,Mathlib/Algebra/BigOperators/Ring.lean,Mathlib/Algebra/GCDMonoid/Finset.lean,Mathlib/Algebra/GCDMonoid/Multiset.lean,Mathlib/Algebra/Group/Subgroup/Finite.lean,Mathlib/Algebra/GroupWithZero/WithZero.lean,Mathlib/Algebra/Lie/Submodule.lean,Mathlib/Algebra/Lie/Weights/Basic.lean,Mathlib/Algebra/Module/BigOperators.lean,Mathlib/Algebra/MvPolynomial/Basic.lean,Mathlib/Algebra/MvPolynomial/Derivation.lean,Mathlib/Algebra/MvPolynomial/Variables.lean,Mathlib/Algebra/Order/ToIntervalMod.lean,Mathlib/Algebra/Polynomial/BigOperators.lean,Mathlib/Algebra/Polynomial/Degree/Lemmas.lean,Mathlib/Algebra/Polynomial/Derivative.lean,Mathlib/Algebra/Polynomial/Eval.lean,Mathlib/Algebra/Polynomial/Induction.lean,Mathlib/Algebra/Polynomial/Module/Basic.lean,Mathlib/Algebra/Polynomial/PartialFractions.lean,Mathlib/Algebra/Polynomial/Smeval.lean,Mathlib/Algebra/Tropical/BigOperators.lean,Mathlib/AlgebraicTopology/DoldKan/NCompGamma.lean,Mathlib/AlgebraicTopology/SimplexCategory.lean,Mathlib/AlgebraicTopology/SplitSimplicialObject.lean,Mathlib/Analysis/Analytic/Constructions.lean,Mathlib/Analysis/Asymptotics/Asymptotics.lean,Mathlib/Analysis/BoxIntegral/Basic.lean,Mathlib/Analysis/BoxIntegral/Partition/Additive.lean,Mathlib/Analysis/BoxIntegral/Partition/Split.lean,Mathlib/Analysis/Calculus/ContDiff/Basic.lean,Mathlib/Analysis/Calculus/ContDiff/Bounds.lean,Mathlib/Analysis/Calculus/Deriv/Polynomial.lean,Mathlib/Analysis/Convex/Combination.lean,Mathlib/Analysis/Convex/Exposed.lean,Mathlib/Analysis/Fourier/AddCircle.lean,Mathlib/Analysis/NormedSpace/Exponential.lean,Mathlib/Analysis/NormedSpace/Multilinear/Basic.lean,Mathlib/Analysis/SpecialFunctions/Complex/Arg.lean,Mathlib/Analysis/SpecialFunctions/Complex/Circle.lean,Mathlib/Analysis/SpecialFunctions/Log/Base.lean,Mathlib/Analysis/SpecialFunctions/PolynomialExp.lean,Mathlib/Analysis/SpecialFunctions/Pow/NNReal.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Angle.lean,Mathlib/CategoryTheory/Filtered/Basic.lean,Mathlib/CategoryTheory/Subobject/Lattice.lean,Mathlib/Combinatorics/Additive/PluenneckeRuzsa.lean,Mathlib/Combinatorics/SetFamily/Compression/Down.lean,Mathlib/Combinatorics/SetFamily/FourFunctions.lean,Mathlib/Combinatorics/SetFamily/HarrisKleitman.lean,Mathlib/Computability/Reduce.lean,Mathlib/Data/DFinsupp/Basic.lean,Mathlib/Data/DFinsupp/WellFounded.lean,Mathlib/Data/Finset/Basic.lean,Mathlib/Data/Finset/Fold.lean,Mathlib/Data/Finset/Lattice.lean,Mathlib/Data/Finset/NAry.lean,Mathlib/Data/Fintype/Sum.lean,Mathlib/Data/Multiset/Antidiagonal.lean,Mathlib/Data/Multiset/Basic.lean,Mathlib/Data/Multiset/Bind.lean,Mathlib/Data/Multiset/Fold.lean,Mathlib/Data/Multiset/Lattice.lean,Mathlib/Data/Multiset/Pi.lean,Mathlib/Data/Multiset/Powerset.lean,Mathlib/Data/Multiset/Sections.lean,Mathlib/Data/Nat/Choose/Multinomial.lean,Mathlib/Data/Nat/PartENat.lean,Mathlib/Data/Quot.lean,Mathlib/Data/Set/Pointwise/BigOperators.lean,Mathlib/FieldTheory/IntermediateField.lean,Mathlib/FieldTheory/IsAlgClosed/AlgebraicClosure.lean,Mathlib/Geometry/Manifold/Algebra/Monoid.lean,Mathlib/Geometry/RingedSpace/Basic.lean,Mathlib/Geometry/RingedSpace/OpenImmersion.lean,Mathlib/Geometry/RingedSpace/PresheafedSpace/Gluing.lean,Mathlib/GroupTheory/Coset.lean,Mathlib/GroupTheory/NoncommPiCoprod.lean,Mathlib/GroupTheory/Perm/Cycle/Type.lean,Mathlib/LinearAlgebra/Determinant.lean,Mathlib/LinearAlgebra/Eigenspace/Basic.lean,Mathlib/LinearAlgebra/FiniteDimensional.lean,Mathlib/LinearAlgebra/LinearIndependent.lean,Mathlib/LinearAlgebra/Matrix/Determinant/Basic.lean,Mathlib/LinearAlgebra/Multilinear/Basic.lean,Mathlib/LinearAlgebra/Orientation.lean,Mathlib/LinearAlgebra/Projectivization/Basic.lean,Mathlib/LinearAlgebra/Ray.lean,Mathlib/LinearAlgebra/TensorProduct/Basic.lean,Mathlib/Logic/Hydra.lean,Mathlib/MeasureTheory/Function/ConditionalExpectation/Basic.lean,Mathlib/MeasureTheory/Function/L1Space.lean,Mathlib/MeasureTheory/Function/SimpleFunc.lean,Mathlib/MeasureTheory/Integral/Lebesgue.lean,Mathlib/MeasureTheory/Integral/Marginal.lean,Mathlib/MeasureTheory/Integral/MeanInequalities.lean,Mathlib/MeasureTheory/Integral/SetIntegral.lean,Mathlib/MeasureTheory/Measure/AddContent.lean |
140 |
14 |
['FR-vdash-bot', 'YaelDillies', 'eric-wieser', 'github-actions', 'leanprover-community-mathlib4-bot', 'urkud'] |
nobody |
146-63912 4 months ago |
432-77838 1 year ago |
4-46495 4 days |
15099 |
joelriou author:joelriou |
feat(CategoryTheory/Sites): the Mayer-Vietoris long exact sequence in sheaf cohomology |
In this PR, we obtain the long exact Mayer-Vietoris sequence in sheaf cohomology `... ⟶ H^n₀(S.X₄, F) ⟶ H^n₀(S.X₂, F) ⊞ H^n₀(S.X₃, F) ⟶ H^n₀(S.X₁, F) ⟶ H^n₁(S.X₄, F) ⟶ ...` when `n₀ + 1 = n₁`. It is attached to any "Mayer-Vietoris square", which includes the typical case of a covering by two open subsets in a topological space. (This API shall also apply to the case of Nisnevich distinguished squares of schemes.)
---
- [x] depends on: #15770
- [x] depends on: #14793
- [x] depends on: #14515
- [x] depends on: #15092
- [x] depends on: #15053
- [x] depends on: #14867
- [x] depends on: #14959
- [x] depends on: #14957
[](https://gitpod.io/from-referrer/)
|
t-category-theory
merge-conflict
WIP
|
348/4 |
Mathlib.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/Basic.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/Biprod.lean,Mathlib/CategoryTheory/Preadditive/Opposite.lean,Mathlib/CategoryTheory/Shift/Basic.lean,Mathlib/CategoryTheory/Shift/ShiftedHom.lean,Mathlib/CategoryTheory/Sites/SheafCohomology/Basic.lean,Mathlib/CategoryTheory/Sites/SheafCohomology/MayerVietoris.lean |
8 |
n/a |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
144-7359 4 months ago |
unknown |
unknown |
23859 |
urkud author:urkud |
feat(Topology/../Order/Field): generalize to `Semifield` |
.. from a linear ordered field to a linear ordered semifield---
- [ ] depends on: #23857
[](https://gitpod.io/from-referrer/)
|
t-topology
merge-conflict
|
245/219 |
Mathlib/Algebra/Order/Group/Pointwise/Interval.lean,Mathlib/Analysis/BoxIntegral/Box/SubboxInduction.lean,Mathlib/Topology/Algebra/Order/Field.lean,Mathlib/Topology/Order/Basic.lean |
4 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
144-3335 4 months ago |
144-3338 4 months ago |
0-265 4 minutes |
23810 |
b-reinke author:b-reinke |
chore(Order/Interval): generalize succ/pred lemmas to partial orders |
Many lemmas in `Mathlib/Order/Interval/Set/SuccPred.lean`and `Mathlib/Order/Interval/Finset/SuccPred.lean` also work for partial orders. They are generalized in this PR by introducing different sections for `PartialOrder` and `LinearOrder` assumptions in the respective files.
---
[](https://gitpod.io/from-referrer/)
|
t-order
merge-conflict
|
231/89 |
Mathlib/Order/Interval/Finset/SuccPred.lean,Mathlib/Order/Interval/Set/SuccPred.lean |
2 |
2 |
['github-actions', 'leanprover-community-bot-assistant'] |
nobody |
141-66510 4 months ago |
141-66512 4 months ago |
16-29623 16 days |
24285 |
madvorak author:madvorak |
chore(Algebra/*-{Category,Homology}): remove unnecessary universe variables |
Discussions:
https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Call.20for.20help.3A.20technical.2F.20organisational.20debt/with/513620128
https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Algebra.20and.20.60Type*.60/with/513558902
https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Task.2026.3A.20Replace.20Type.20u.20by.20Type*.20wherever.20possible/with/513592993
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
label:t-algebra$ |
542/916 |
Mathlib/Algebra/AddTorsor/Basic.lean,Mathlib/Algebra/Algebra/Defs.lean,Mathlib/Algebra/Algebra/Equiv.lean,Mathlib/Algebra/Algebra/Field.lean,Mathlib/Algebra/Algebra/Hom.lean,Mathlib/Algebra/Algebra/Operations.lean,Mathlib/Algebra/Algebra/Spectrum/Basic.lean,Mathlib/Algebra/Algebra/Subalgebra/Lattice.lean,Mathlib/Algebra/Algebra/Subalgebra/Tower.lean,Mathlib/Algebra/Algebra/Tower.lean,Mathlib/Algebra/Central/Basic.lean,Mathlib/Algebra/Central/Defs.lean,Mathlib/Algebra/Central/TensorProduct.lean,Mathlib/Algebra/CharP/Pi.lean,Mathlib/Algebra/CharP/Quotient.lean,Mathlib/Algebra/CharP/Subring.lean,Mathlib/Algebra/DirectSum/Algebra.lean,Mathlib/Algebra/DirectSum/Basic.lean,Mathlib/Algebra/DirectSum/Finsupp.lean,Mathlib/Algebra/DirectSum/Module.lean,Mathlib/Algebra/EuclideanDomain/Basic.lean,Mathlib/Algebra/EuclideanDomain/Defs.lean,Mathlib/Algebra/Field/Basic.lean,Mathlib/Algebra/Field/Defs.lean,Mathlib/Algebra/Field/IsField.lean,Mathlib/Algebra/Field/MinimalAxioms.lean,Mathlib/Algebra/Field/Subfield/Basic.lean,Mathlib/Algebra/Field/Subfield/Defs.lean,Mathlib/Algebra/FreeNonUnitalNonAssocAlgebra.lean,Mathlib/Algebra/Group/Conj.lean,Mathlib/Algebra/Group/Defs.lean,Mathlib/Algebra/Group/Equiv/Finite.lean,Mathlib/Algebra/Group/Ext.lean,Mathlib/Algebra/Group/Hom/End.lean,Mathlib/Algebra/Group/Hom/Instances.lean,Mathlib/Algebra/Group/Invertible/Basic.lean,Mathlib/Algebra/Group/Invertible/Defs.lean,Mathlib/Algebra/Group/Pi/Basic.lean,Mathlib/Algebra/Group/Pi/Lemmas.lean,Mathlib/Algebra/Group/TypeTags/Basic.lean,Mathlib/Algebra/Group/TypeTags/Finite.lean,Mathlib/Algebra/Group/TypeTags/Hom.lean,Mathlib/Algebra/Group/Units/Basic.lean,Mathlib/Algebra/Group/Units/Defs.lean,Mathlib/Algebra/Group/Units/Hom.lean,Mathlib/Algebra/Group/WithOne/Basic.lean,Mathlib/Algebra/Group/WithOne/Defs.lean,Mathlib/Algebra/GroupWithZero/Action/Pi.lean,Mathlib/Algebra/GroupWithZero/Defs.lean,Mathlib/Algebra/GroupWithZero/Invertible.lean,Mathlib/Algebra/GroupWithZero/NeZero.lean,Mathlib/Algebra/Lie/Abelian.lean,Mathlib/Algebra/Lie/Basic.lean,Mathlib/Algebra/Lie/CartanMatrix.lean,Mathlib/Algebra/Lie/CartanSubalgebra.lean,Mathlib/Algebra/Lie/Character.lean,Mathlib/Algebra/Lie/Classical.lean,Mathlib/Algebra/Lie/DirectSum.lean,Mathlib/Algebra/Lie/Free.lean,Mathlib/Algebra/Lie/Ideal.lean,Mathlib/Algebra/Lie/IdealOperations.lean,Mathlib/Algebra/Lie/Matrix.lean,Mathlib/Algebra/Lie/Nilpotent.lean,Mathlib/Algebra/Lie/NonUnitalNonAssocAlgebra.lean,Mathlib/Algebra/Lie/OfAssociative.lean,Mathlib/Algebra/Lie/Quotient.lean,Mathlib/Algebra/Lie/SkewAdjoint.lean,Mathlib/Algebra/Lie/Solvable.lean,Mathlib/Algebra/Lie/Subalgebra.lean,Mathlib/Algebra/Lie/Submodule.lean,Mathlib/Algebra/Lie/TensorProduct.lean,Mathlib/Algebra/Lie/UniversalEnveloping.lean,Mathlib/Algebra/Module/Basic.lean,Mathlib/Algebra/Module/CharacterModule.lean,Mathlib/Algebra/Module/DedekindDomain.lean,Mathlib/Algebra/Module/Defs.lean,Mathlib/Algebra/Module/End.lean,Mathlib/Algebra/Module/Equiv/Opposite.lean,Mathlib/Algebra/Module/Lattice.lean,Mathlib/Algebra/Module/LinearMap/Basic.lean,Mathlib/Algebra/Module/LinearMap/Defs.lean,Mathlib/Algebra/Module/LinearMap/End.lean,Mathlib/Algebra/Module/LocalizedModule/Basic.lean,Mathlib/Algebra/Module/MinimalAxioms.lean,Mathlib/Algebra/Module/NatInt.lean,Mathlib/Algebra/Module/Opposite.lean,Mathlib/Algebra/Module/Pi.lean,Mathlib/Algebra/Module/Presentation/Differentials.lean,Mathlib/Algebra/Module/Presentation/Tensor.lean,Mathlib/Algebra/Module/Rat.lean,Mathlib/Algebra/Module/RingHom.lean,Mathlib/Algebra/Module/Submodule/Basic.lean,Mathlib/Algebra/Module/Torsion.lean,Mathlib/Algebra/MonoidAlgebra/Basic.lean,Mathlib/Algebra/MonoidAlgebra/Defs.lean,Mathlib/Algebra/MonoidAlgebra/Support.lean,Mathlib/Algebra/MvPolynomial/Basic.lean,Mathlib/Algebra/MvPolynomial/CommRing.lean,Mathlib/Algebra/MvPolynomial/Degrees.lean,Mathlib/Algebra/MvPolynomial/Equiv.lean |
182 |
22 |
['erdOne', 'github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'madvorak', 'mattrobball'] |
nobody |
141-55207 4 months ago |
141-55208 4 months ago |
2-12022 2 days |
8370 |
eric-wieser author:eric-wieser |
refactor(Analysis/NormedSpace/Exponential): remove the `𝕂` argument from `exp` |
This argument is still needed for almost all the lemmas, which means it can longer be found by unification.
We keep around `expSeries 𝕂 A`, as it's needed for talking about the radius of convergence over different base fields.
This is a prerequisite for #8372, as we can't merge the functions until they have the same interface.\
Zulip thread: [#mathlib4 > Real.exp @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Real.2Eexp/near/401602245)
---
[](https://gitpod.io/from-referrer/)
This is started from the mathport output on https://github.com/leanprover-community/mathlib/pull/19244 |
awaiting-zulip
t-analysis
merge-conflict
|
432/387 |
Mathlib/Analysis/CStarAlgebra/Exponential.lean,Mathlib/Analysis/CStarAlgebra/Spectrum.lean,Mathlib/Analysis/Normed/Algebra/Exponential.lean,Mathlib/Analysis/Normed/Algebra/MatrixExponential.lean,Mathlib/Analysis/Normed/Algebra/QuaternionExponential.lean,Mathlib/Analysis/Normed/Algebra/Spectrum.lean,Mathlib/Analysis/Normed/Algebra/TrivSqZeroExt.lean,Mathlib/Analysis/NormedSpace/DualNumber.lean,Mathlib/Analysis/SpecialFunctions/ContinuousFunctionalCalculus/ExpLog.lean,Mathlib/Analysis/SpecialFunctions/Exponential.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Series.lean |
11 |
29 |
['YaelDillies', 'eric-wieser', 'girving', 'github-actions', 'j-loreaux', 'kbuzzard', 'leanprover-community-bot-assistant', 'urkud'] |
nobody |
141-36137 4 months ago |
152-64767 4 months ago |
29-60989 29 days |
14931 |
eric-wieser author:eric-wieser |
feat: volume of a simplex |
---
[](https://gitpod.io/from-referrer/)
|
t-euclidean-geometry
merge-conflict
|
207/0 |
Mathlib/Geometry/Euclidean/Basic.lean,Mathlib/Geometry/Euclidean/Circumcenter.lean,Mathlib/Geometry/Euclidean/Volume.lean |
3 |
3 |
['eric-wieser', 'github-actions', 'leanprover-community-bot-assistant'] |
nobody |
139-67664 4 months ago |
139-67666 4 months ago |
0-0 0 seconds |
22583 |
imathwy author:imathwy |
feat: affinespace homeomorphism |
There exists a homeomorphism (a continuous bijection with a continuous inverse) between an affine subspace s of a vector space V over a field 𝕜 and its direction s.direction , given a chosen point z ∈ s .
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
awaiting-author
label:t-algebra$ |
64/2 |
Mathlib/Analysis/Normed/Group/AddTorsor.lean,Mathlib/LinearAlgebra/AffineSpace/ContinuousAffineEquiv.lean,Mathlib/Topology/Algebra/ConstMulAction.lean,Mathlib/Topology/Algebra/MulAction.lean |
4 |
6 |
['JovanGerb', 'eric-wieser', 'github-actions', 'grunweg'] |
nobody |
139-65382 4 months ago |
180-24075 5 months ago |
0-18122 5 hours |
24243 |
Timeroot author:Timeroot |
feat(Analysis/Calculus/FDeriv): Fderiv on torsors |
Experiment to see how this goes for now, see [Zulip discussion](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Upgrade.20.60fderiv.60.20to.20.60AddTorsor.60)
---
[](https://gitpod.io/from-referrer/)
|
t-analysis
merge-conflict
|
539/447 |
Mathlib/Algebra/AddTorsor/Defs.lean,Mathlib/Analysis/Calculus/Deriv/Basic.lean,Mathlib/Analysis/Calculus/Deriv/Prod.lean,Mathlib/Analysis/Calculus/Deriv/Slope.lean,Mathlib/Analysis/Calculus/FDeriv/Add.lean,Mathlib/Analysis/Calculus/FDeriv/Basic.lean,Mathlib/Analysis/Calculus/FDeriv/Bilinear.lean,Mathlib/Analysis/Calculus/FDeriv/Equiv.lean,Mathlib/Analysis/Calculus/FDeriv/Linear.lean,Mathlib/Analysis/Calculus/FDeriv/Measurable.lean,Mathlib/Analysis/Calculus/FDeriv/Mul.lean,Mathlib/Analysis/Calculus/FDeriv/Symmetric.lean,Mathlib/Analysis/Calculus/Gradient/Basic.lean,Mathlib/Analysis/Calculus/LineDeriv/Basic.lean,Mathlib/Analysis/Calculus/LocalExtr/Basic.lean,Mathlib/Analysis/Calculus/ParametricIntegral.lean,Mathlib/Analysis/Calculus/Rademacher.lean,Mathlib/Analysis/Calculus/TangentCone.lean,Mathlib/Analysis/Calculus/UniformLimitsDeriv.lean,Mathlib/Analysis/Complex/Periodic.lean,Mathlib/Analysis/Complex/RealDeriv.lean,Mathlib/Analysis/MellinTransform.lean,Mathlib/Analysis/Normed/Group/Uniform.lean,Mathlib/Analysis/Normed/Module/Basic.lean,Mathlib/Analysis/SpecialFunctions/ExpDeriv.lean,Mathlib/Analysis/SpecialFunctions/Exponential.lean,Mathlib/Analysis/SpecialFunctions/Gamma/Deriv.lean,Mathlib/Analysis/SpecialFunctions/Pow/Deriv.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/EulerSineProd.lean,Mathlib/Geometry/Manifold/IntegralCurve/Transform.lean,Mathlib/Geometry/Manifold/IsManifold/Basic.lean,Mathlib/Geometry/Manifold/MFDeriv/Basic.lean,Mathlib/Geometry/Manifold/MFDeriv/SpecificFunctions.lean,Mathlib/NumberTheory/EulerProduct/ExpLog.lean,Mathlib/NumberTheory/Harmonic/GammaDeriv.lean,Mathlib/NumberTheory/LSeries/Nonvanishing.lean,MathlibTest/Recall.lean |
37 |
3 |
['github-actions', 'leanprover-community-bot-assistant'] |
nobody |
138-48520 4 months ago |
138-48521 4 months ago |
0-0 0 seconds |
24322 |
mattrobball author:mattrobball |
chore: merge repeated `Type*` binders |
Per the discussion on [Zulip](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Task.2026.3A.20Replace.20Type.20u.20by.20Type*.20wherever.20possible), this PR merges `(A : Type*) (B : Type u)` into `(A B : Type*)` and similarly for `{}`.
NOTE: the Python script used it currently in the `/scripts` folder. It is there for inspection and should be removed before merging this PR.
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict
awaiting-author
|
685/591 |
Archive/Imo/Imo2019Q2.lean,Archive/Wiedijk100Theorems/HeronsFormula.lean,Mathlib/Algebra/AddTorsor/Basic.lean,Mathlib/Algebra/AddTorsor/Defs.lean,Mathlib/Algebra/Algebra/Basic.lean,Mathlib/Algebra/Algebra/Pi.lean,Mathlib/Algebra/Algebra/Subalgebra/Pointwise.lean,Mathlib/Algebra/Algebra/Unitization.lean,Mathlib/Algebra/BigOperators/Fin.lean,Mathlib/Algebra/BigOperators/Finsupp/Basic.lean,Mathlib/Algebra/Category/ModuleCat/ChangeOfRings.lean,Mathlib/Algebra/DirectSum/Internal.lean,Mathlib/Algebra/FreeMonoid/Basic.lean,Mathlib/Algebra/Group/Action/Defs.lean,Mathlib/Algebra/Group/Action/Faithful.lean,Mathlib/Algebra/Group/Action/Sigma.lean,Mathlib/Algebra/Group/Hom/Basic.lean,Mathlib/Algebra/Group/Hom/Defs.lean,Mathlib/Algebra/Group/InjSurj.lean,Mathlib/Algebra/Group/Invertible/Basic.lean,Mathlib/Algebra/Group/Prod.lean,Mathlib/Algebra/Group/Subgroup/Basic.lean,Mathlib/Algebra/Group/Subgroup/Ker.lean,Mathlib/Algebra/Group/Submonoid/Basic.lean,Mathlib/Algebra/Group/Submonoid/Defs.lean,Mathlib/Algebra/Group/Submonoid/Membership.lean,Mathlib/Algebra/Group/Submonoid/MulAction.lean,Mathlib/Algebra/Group/Submonoid/Operations.lean,Mathlib/Algebra/Group/Subsemigroup/Basic.lean,Mathlib/Algebra/Group/Subsemigroup/Defs.lean,Mathlib/Algebra/Group/Subsemigroup/Operations.lean,Mathlib/Algebra/Group/Support.lean,Mathlib/Algebra/Group/Units/Defs.lean,Mathlib/Algebra/Module/Equiv/Basic.lean,Mathlib/Algebra/Module/Equiv/Defs.lean,Mathlib/Algebra/Module/LinearMap/Defs.lean,Mathlib/Algebra/Module/LinearMap/Prod.lean,Mathlib/Algebra/Module/Prod.lean,Mathlib/Algebra/Module/Submodule/EqLocus.lean,Mathlib/Algebra/Module/Submodule/Equiv.lean,Mathlib/Algebra/Module/Submodule/Ker.lean,Mathlib/Algebra/Module/Submodule/LinearMap.lean,Mathlib/Algebra/Module/Submodule/Map.lean,Mathlib/Algebra/Module/Submodule/Pointwise.lean,Mathlib/Algebra/Module/Submodule/Range.lean,Mathlib/Algebra/MonoidAlgebra/Grading.lean,Mathlib/Algebra/MonoidAlgebra/MapDomain.lean,Mathlib/Algebra/MonoidAlgebra/ToDirectSum.lean,Mathlib/Algebra/MvPolynomial/Basic.lean,Mathlib/Algebra/MvPolynomial/Comap.lean,Mathlib/Algebra/MvPolynomial/Monad.lean,Mathlib/Algebra/Notation/Prod.lean,Mathlib/Algebra/Order/Quantale.lean,Mathlib/Algebra/Prime/Lemmas.lean,Mathlib/Algebra/Quandle.lean,Mathlib/Algebra/QuaternionBasis.lean,Mathlib/Algebra/Ring/CompTypeclasses.lean,Mathlib/Algebra/Ring/Hom/Defs.lean,Mathlib/Algebra/SkewMonoidAlgebra/Basic.lean,Mathlib/Algebra/Star/Module.lean,Mathlib/Algebra/TrivSqZeroExt.lean,Mathlib/Algebra/Vertex/HVertexOperator.lean,Mathlib/Algebra/Vertex/VertexOperator.lean,Mathlib/Analysis/Analytic/Composition.lean,Mathlib/Analysis/Asymptotics/Defs.lean,Mathlib/Analysis/Asymptotics/Lemmas.lean,Mathlib/Analysis/Asymptotics/Theta.lean,Mathlib/Analysis/CStarAlgebra/CStarMatrix.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Integral.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Order.lean,Mathlib/Analysis/Calculus/ContDiff/Bounds.lean,Mathlib/Analysis/Calculus/Deriv/Mul.lean,Mathlib/Analysis/Calculus/FDeriv/Mul.lean,Mathlib/Analysis/Calculus/FormalMultilinearSeries.lean,Mathlib/Analysis/Convex/Cone/Proper.lean,Mathlib/Analysis/Convex/EGauge.lean,Mathlib/Analysis/Convex/Exposed.lean,Mathlib/Analysis/InnerProductSpace/Adjoint.lean,Mathlib/Analysis/InnerProductSpace/Defs.lean,Mathlib/Analysis/InnerProductSpace/LinearMap.lean,Mathlib/Analysis/InnerProductSpace/Orthonormal.lean,Mathlib/Analysis/InnerProductSpace/PiL2.lean,Mathlib/Analysis/InnerProductSpace/WeakOperatorTopology.lean,Mathlib/Analysis/LocallyConvex/WeakOperatorTopology.lean,Mathlib/Analysis/Normed/Affine/Isometry.lean,Mathlib/Analysis/Normed/Algebra/Basic.lean,Mathlib/Analysis/Normed/Algebra/Spectrum.lean,Mathlib/Analysis/Normed/Lp/lpSpace.lean,Mathlib/Analysis/Normed/Module/Basic.lean,Mathlib/Analysis/Normed/Module/FiniteDimension.lean,Mathlib/Analysis/Normed/Ring/InfiniteSum.lean,Mathlib/Analysis/Normed/Ring/Lemmas.lean,Mathlib/Analysis/NormedSpace/ConformalLinearMap.lean,Mathlib/Analysis/NormedSpace/ENormedSpace.lean,Mathlib/Analysis/NormedSpace/OperatorNorm/Bilinear.lean,Mathlib/Analysis/Seminorm.lean,Mathlib/Analysis/SpecialFunctions/ContinuousFunctionalCalculus/ExpLog.lean,Mathlib/Analysis/SpecificLimits/Basic.lean,Mathlib/CategoryTheory/Action/Concrete.lean,Mathlib/CategoryTheory/GradedObject.lean |
343 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'urkud'] |
nobody |
138-47998 4 months ago |
138-48000 4 months ago |
2-7052 2 days |
23138 |
grunweg author:grunweg |
feat: (unoriented) bordism groups |
We define the unoriented bordism group of a topological space and prove that it is an abelian group:
we don't prove transitivity of bordisms yet, as that requires the collar neighbourhood theorem and gluing of smooth manifolds, which are both not in mathlib and a sizable piece of work.
---
This PR is not ready for review yet; I'm merely opening this to track this branch' state better. In particular, this PR depends on several preliminary PRs:
- depends on: #15906 for defining singular n-manifolds
- depends on: #23040: define immersions and smooth embeddings: in finite dimensions, these are easy to describe; for mathlib, we will want a correct definition for e.g. Banach manifolds also.
- depends on: #22059 defines manifolds with smooth boundary. That PR has two open dependencies; one is slowly getting merged, that other has a few sorries I still need to prove (not difficult).
- depends on: #22874 for some constructions
- defining unoriented bordisms, and proving some basic constructions about them: will be another PR
[](https://gitpod.io/from-referrer/)
|
t-differential-geometry
merge-conflict
WIP
|
1316/3 |
Mathlib.lean,Mathlib/Geometry/Manifold/Bordisms.lean,Mathlib/Geometry/Manifold/Diffeomorph.lean,Mathlib/Geometry/Manifold/HasSmoothBoundary.lean,Mathlib/Geometry/Manifold/Instances/Real.lean,Mathlib/Geometry/Manifold/IsManifold/Basic.lean,Mathlib/Geometry/Manifold/MFDeriv/SpecificFunctions.lean |
7 |
0 |
[] |
nobody |
137-82892 4 months ago |
175-59173 5 months ago |
0-1 1 second |
23593 |
erdOne author:erdOne |
feat(AlgebraicGeometry): the tilde construction is functorial |
---
[](https://gitpod.io/from-referrer/)
|
t-algebraic-geometry
merge-conflict
awaiting-author
|
95/38 |
Mathlib/AlgebraicGeometry/Modules/Sheaf.lean,Mathlib/AlgebraicGeometry/Modules/Tilde.lean |
2 |
4 |
['chrisflav', 'github-actions', 'leanprover-community-bot-assistant'] |
nobody |
137-82578 4 months ago |
137-82580 4 months ago |
0-71091 19 hours |
21065 |
eric-wieser author:eric-wieser |
feat: generalize `tangentConeAt.lim_zero` to TVS |
... and then adjust the `variable`s down the rest of the file to make use of the generality.
There are two key lemmas that this does not generalize, which would probably unlock the rest of the file:
* `subset_tangentCone_prod_left` (and `_right`)
* `zero_mem_tangentCone`
---
- [ ] depends on: #20859
[](https://gitpod.io/from-referrer/)
|
t-analysis
merge-conflict
WIP
|
55/28 |
Mathlib/Analysis/Calculus/TangentCone.lean |
1 |
16 |
['ADedecker', 'eric-wieser', 'github-actions', 'j-loreaux', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'urkud'] |
nobody |
137-74982 4 months ago |
137-74984 4 months ago |
23-20319 23 days |
22721 |
grunweg author:grunweg |
chore(MeasureTheory/Function/LpSeminorm/Basic): generalise more results to enorm classes |
Done for the Carleson project.
---
- depends on #22708
[](https://gitpod.io/from-referrer/)
|
carleson
t-measure-probability
merge-conflict
WIP
|
134/10 |
Mathlib/MeasureTheory/Function/LpSeminorm/Basic.lean |
1 |
2 |
['github-actions', 'leanprover-community-bot-assistant'] |
nobody |
136-67650 4 months ago |
136-67652 4 months ago |
0-6 6 seconds |
24354 |
grunweg author:grunweg |
chore(HasFiniteIntegral): rename three lemmas |
Discovered in #24343.
---
- [ ] depends on: #24343 (to avoid merge conflicts)
[](https://gitpod.io/from-referrer/)
|
t-measure-probability
merge-conflict
|
108/30 |
Mathlib/MeasureTheory/Function/L1Space/HasFiniteIntegral.lean |
1 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
136-59611 4 months ago |
136-59612 4 months ago |
0-4604 1 hour |
23791 |
SEU-Prime author:SEU-Prime |
Create AmiceTrans.lean |
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-number-theory
merge-conflict
WIP
|
2963/0 |
Mathlib.lean,Mathlib/Analysis/Normed/Ring/Lemmas2.lean,Mathlib/NumberTheory/Padics/AmiceTrans.lean,Mathlib/NumberTheory/Padics/PSAC.lean,Mathlib/NumberTheory/Padics/PSAC2.lean,Mathlib/NumberTheory/Padics/PSAC3.lean,Mathlib/NumberTheory/Padics/PiGammainPS.lean,Mathlib/NumberTheory/Padics/PsiandVar.lean,Mathlib/RingTheory/AdicCompletion/Lemma.lean,Mathlib/RingTheory/PowerSeries/Comp.lean,Mathlib/Topology/ContinuousMap/ZeroAtBot.lean |
11 |
3 |
['SEU-Prime', 'github-actions', 'leanprover-community-bot-assistant'] |
nobody |
136-20531 4 months ago |
142-85937 4 months ago |
0-0 0 seconds |
24091 |
mattrobball author:mattrobball |
test |
|
merge-conflict |
97/46 |
Mathlib/Algebra/Field/Defs.lean,Mathlib/Analysis/Asymptotics/Lemmas.lean,Mathlib/Analysis/LocallyConvex/Basic.lean,Mathlib/Analysis/Normed/Affine/AddTorsor.lean,Mathlib/Analysis/Normed/Module/Basic.lean,Mathlib/Analysis/Normed/Module/Span.lean,Mathlib/Analysis/Normed/MulAction.lean,Mathlib/Analysis/NormedSpace/Pointwise.lean,Mathlib/Dynamics/BirkhoffSum/NormedSpace.lean,Mathlib/MeasureTheory/Function/LpSeminorm/Basic.lean,Mathlib/Topology/ContinuousMap/Compact.lean,Mathlib/Topology/MetricSpace/Holder.lean,Mathlib/Topology/MetricSpace/HolderNorm.lean,docs/overview.yaml,docs/undergrad.yaml |
15 |
5 |
['github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'mattrobball'] |
nobody |
136-9949 4 months ago |
136-9951 4 months ago |
0-0 0 seconds |
14731 |
adomani author:adomani |
feat: the repeated typeclass assumption linter |
[#mathlib4 > recyclable variables @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/recyclable.20variables/near/451167963) also [#mathlib4 > Normed modules @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Normed.20modules/near/512242167)
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-linter
merge-conflict
WIP
|
178/0 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter.lean,Mathlib/Tactic/Linter/DependentTypeclass.lean,MathlibTest/DependentTypeclass.lean |
5 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mattrobball'] |
nobody |
135-72889 4 months ago |
148-3891 4 months ago |
0-109 1 minute |
24140 |
mattrobball author:mattrobball |
test |
|
merge-conflict |
176/91 |
Mathlib/Algebra/Group/Defs.lean,Mathlib/Algebra/GroupWithZero/Defs.lean,Mathlib/Algebra/Ring/Defs.lean,Mathlib/AlgebraicGeometry/AffineSpace.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Affine.lean,Mathlib/Analysis/CStarAlgebra/Classes.lean,Mathlib/Data/Complex/Module.lean,Mathlib/LinearAlgebra/Matrix/Charpoly/Coeff.lean,Mathlib/NumberTheory/NumberField/ProductFormula.lean,Mathlib/RingTheory/Algebraic/Integral.lean,Mathlib/RingTheory/LaurentSeries.lean,Mathlib/RingTheory/Localization/Integral.lean,Mathlib/RingTheory/RingHom/Unramified.lean,Mathlib/RingTheory/Spectrum/Prime/ChevalleyComplexity.lean,Mathlib/RingTheory/Valuation/Basic.lean,Mathlib/RingTheory/Valuation/ValuationSubring.lean,Mathlib/Topology/Algebra/Valued/WithVal.lean |
17 |
5 |
['github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'mattrobball'] |
nobody |
135-71352 4 months ago |
135-71354 4 months ago |
0-0 0 seconds |
13649 |
FR-vdash-bot author:FR-vdash-bot |
chore: redefine `Nat.div2` `Nat.bodd` |
The new definitions are faster than the old ones. `Nat.binaryRec` will be moved to batteries (https://github.com/leanprover-community/batteries/pull/799) or core (https://github.com/leanprover/lean4/pull/3756), so relevant contents are moved to a new file temporarily.
---
- [x] depends on: #15567
- [x] depends on: #19666
[](https://gitpod.io/from-referrer/)
|
merge-conflict |
63/88 |
Mathlib/Computability/Primrec.lean,Mathlib/Data/Int/Bitwise.lean,Mathlib/Data/Nat/Bits.lean,Mathlib/Data/Nat/Bitwise.lean,Mathlib/Data/Nat/Size.lean,Mathlib/Logic/Denumerable.lean,Mathlib/Logic/Encodable/Basic.lean,Mathlib/Logic/Equiv/Nat.lean |
8 |
15 |
['FR-vdash-bot', 'digama0', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'urkud'] |
digama0 assignee:digama0 |
133-38757 4 months ago |
133-38759 4 months ago |
87-51692 87 days |
22856 |
mattrobball author:mattrobball |
test |
|
merge-conflict |
8/2 |
Mathlib/Algebra/Algebra/Defs.lean,Mathlib/Analysis/Complex/Hadamard.lean,Mathlib/Analysis/RCLike/Inner.lean,Mathlib/FieldTheory/Galois/Profinite.lean |
4 |
5 |
['github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'mattrobball'] |
nobody |
133-26318 4 months ago |
133-26320 4 months ago |
0-0 0 seconds |
23921 |
alreadydone author:alreadydone |
Jyxu/projective trace |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
WIP
label:t-algebra$ |
157/123 |
Mathlib/FieldTheory/CardinalEmb.lean,Mathlib/FieldTheory/Relrank.lean,Mathlib/LinearAlgebra/Contraction.lean,Mathlib/LinearAlgebra/Dual.lean,Mathlib/RingTheory/LocalProperties/Projective.lean |
5 |
1 |
['leanprover-community-bot-assistant'] |
nobody |
133-11534 4 months ago |
133-11534 4 months ago |
0-0 0 seconds |
21252 |
ADedecker author:ADedecker |
feat: redefine uniformly convex normed spaces with filters instead of epsilons |
And conceptualize some proofs.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-topology
merge-conflict
label:t-algebra$ |
301/87 |
Mathlib/Analysis/Convex/Uniform.lean,Mathlib/Analysis/InnerProductSpace/Basic.lean,Mathlib/Order/Basic.lean,Mathlib/Order/Filter/Pointwise.lean,Mathlib/Topology/Algebra/UniformGroup/Defs.lean,Mathlib/Topology/Algebra/UniformMulAction.lean |
6 |
1 |
['github-actions'] |
nobody |
133-11273 4 months ago |
133-11273 4 months ago |
0-0 0 seconds |
19821 |
eric-wieser author:eric-wieser |
feat: add a Qq version of AtomM that groups by type |
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-meta
merge-conflict
WIP
|
332/30 |
Mathlib/Data/Ineq.lean,Mathlib/Tactic/Linarith/Datatypes.lean,Mathlib/Tactic/Linarith/Oracle/SimplexAlgorithm.lean,Mathlib/Tactic/Linarith/Preprocessing.lean,Mathlib/Util/AtomM.lean,Mathlib/Util/Qq.lean |
6 |
1 |
['github-actions'] |
nobody |
133-11086 4 months ago |
133-11086 4 months ago |
0-0 0 seconds |
19520 |
erdOne author:erdOne |
refactor(Algebra/Module): Redefine `LocalizedModule` in terms of `OreLocalization` |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
label:t-algebra$ |
610/493 |
Mathlib.lean,Mathlib/Algebra/Module/LocalizedModule/Basic.lean,Mathlib/AlgebraicGeometry/AffineScheme.lean,Mathlib/AlgebraicGeometry/Modules/Tilde.lean,Mathlib/AlgebraicGeometry/OpenImmersion.lean,Mathlib/GroupTheory/OreLocalization/Basic.lean,Mathlib/RingTheory/Localization/BaseChange.lean,Mathlib/RingTheory/OreLocalization/Basic.lean,Mathlib/RingTheory/OreLocalization/Module.lean,Mathlib/RingTheory/OreLocalization/Ring.lean |
10 |
1 |
['github-actions'] |
nobody |
133-11075 4 months ago |
133-11075 4 months ago |
8-56155 8 days |
19120 |
hrmacbeth author:hrmacbeth |
feat: stop `ring`/`abel` from seeing algebraic operations inside `let`s |
This draft PR illustrates a feature I would like to see in core: a variant of `whnf` which allows particular kinds of reduction, such as zeta-delta reduction, to be turned off. Here it is used to make ring-normalization and abelian-group-normalization a bit more responsive to what (I think) users expect: these normalizations would no longer look inside user-defined lets to see algebraic operations in those expressions.
Note: In Lean/Mathlib 3, `ring` matched for algebraic operations on an algebraic expression `e` itself, not on `← whnfR e`. So mathlib3 `ring` didn't see algebraic operations inside `let`s -- but it also didn't see algebraic operations requiring beta-reduction (like `(fun t ↦ t + 1) x`) or see inside abbreviations.
[Zulip](https://leanprover.zulipchat.com/#narrow/channel/239415-metaprogramming-.2F-tactics/topic/whnf.20variant.20which.20preserves.20let-bindings)
Update: fortuitously, it looks like the new core PR https://github.com/leanprover/lean4/pull/6053 will provide this feature!
---
[](https://gitpod.io/from-referrer/)
|
t-meta
merge-conflict
blocked-by-core-PR
|
137/15 |
Archive/Imo/Imo2006Q3.lean,Archive/Imo/Imo2008Q2.lean,Mathlib.lean,Mathlib/Algebra/ContinuedFractions/Computation/Approximations.lean,Mathlib/Analysis/Analytic/Composition.lean,Mathlib/Analysis/Calculus/FDeriv/Measurable.lean,Mathlib/Analysis/SpecialFunctions/Gamma/BohrMollerup.lean,Mathlib/Analysis/SpecialFunctions/Integrals.lean,Mathlib/Analysis/SpecialFunctions/Stirling.lean,Mathlib/Data/Real/Pi/Irrational.lean,Mathlib/NumberTheory/LSeries/HurwitzZetaOdd.lean,Mathlib/NumberTheory/SumPrimeReciprocals.lean,Mathlib/RingTheory/WittVector/DiscreteValuationRing.lean,Mathlib/Tactic/Abel.lean,Mathlib/Tactic/Polyrith.lean,Mathlib/Tactic/Ring/Basic.lean,Mathlib/Tactic/Ring/RingNF.lean,Mathlib/Topology/MetricSpace/GromovHausdorff.lean,Mathlib/Util/WHNF.lean,MathlibTest/abel.lean,MathlibTest/ring.lean |
21 |
5 |
['JovanGerb', 'github-actions', 'grunweg', 'hrmacbeth'] |
nobody |
133-11066 4 months ago |
133-11066 4 months ago |
0-0 0 seconds |
17069 |
yuma-mizuno author:yuma-mizuno |
chore(CategoryTheory/Functor/Basic): put `simp` at `Functor.id_comp` |
---
[](https://gitpod.io/from-referrer/)
|
t-category-theory
merge-conflict
|
41/30 |
Mathlib/CategoryTheory/Adjunction/Mates.lean,Mathlib/CategoryTheory/Functor/Basic.lean,Mathlib/CategoryTheory/GuitartExact/VerticalComposition.lean,Mathlib/CategoryTheory/Limits/HasLimits.lean,Mathlib/CategoryTheory/Shift/CommShift.lean |
5 |
3 |
['github-actions', 'leanprover-bot', 'yuma-mizuno'] |
nobody |
133-11056 4 months ago |
133-11056 4 months ago |
0-0 0 seconds |
15024 |
mattrobball author:mattrobball |
chore(Algebra.Basic): scope and rename universal `Nat`-algebra and `Int`-algebra instances |
We rename `algebraNat` to `Nat.instAlgebraOfSemiring` and `algebraInt` to `Int.instAlgebraOfRing` to be consistent with existing naming conventions. We also scope them to avoid typeclass search tripping over them unnecessarily.
---
Moves:
- algebraNat -> Nat.instAlgebraOfSemiring
- algebraInt -> Int.instAlgebraOfRing
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
label:t-algebra$ |
178/27 |
Archive/Wiedijk100Theorems/AbelRuffini.lean,Counterexamples/Pseudoelement.lean,Mathlib/Algebra/Algebra/Basic.lean,Mathlib/Algebra/Algebra/Hom.lean,Mathlib/Algebra/Algebra/Subalgebra/Basic.lean,Mathlib/Algebra/Algebra/Subalgebra/Unitization.lean,Mathlib/Algebra/Category/ModuleCat/Injective.lean,Mathlib/Algebra/FreeAlgebra.lean,Mathlib/Algebra/Module/Bimodule.lean,Mathlib/Algebra/Module/Zlattice/Basic.lean,Mathlib/Algebra/MvPolynomial/Counit.lean,Mathlib/Algebra/MvPolynomial/Supported.lean,Mathlib/Algebra/Polynomial/AlgebraMap.lean,Mathlib/Algebra/Polynomial/DenomsClearable.lean,Mathlib/Algebra/Polynomial/UnitTrinomial.lean,Mathlib/Algebra/RingQuot.lean,Mathlib/Analysis/Complex/UpperHalfPlane/Basic.lean,Mathlib/Analysis/Complex/UpperHalfPlane/Metric.lean,Mathlib/Analysis/Complex/UpperHalfPlane/Topology.lean,Mathlib/Data/Matrix/Kronecker.lean,Mathlib/Data/Real/Irrational.lean,Mathlib/FieldTheory/IsAlgClosed/Classification.lean,Mathlib/LinearAlgebra/CliffordAlgebra/Basic.lean,Mathlib/LinearAlgebra/FreeModule/IdealQuotient.lean,Mathlib/LinearAlgebra/FreeProduct/Basic.lean,Mathlib/LinearAlgebra/Matrix/Adjugate.lean,Mathlib/LinearAlgebra/QuadraticForm/Basic.lean,Mathlib/LinearAlgebra/TensorAlgebra/Basic.lean,Mathlib/NumberTheory/ClassNumber/AdmissibleCardPowDegree.lean,Mathlib/NumberTheory/ClassNumber/Finite.lean,Mathlib/NumberTheory/Cyclotomic/Basic.lean,Mathlib/NumberTheory/Cyclotomic/Discriminant.lean,Mathlib/NumberTheory/Cyclotomic/Rat.lean,Mathlib/NumberTheory/FLT/Three.lean,Mathlib/NumberTheory/LegendreSymbol/QuadraticChar/GaussSum.lean,Mathlib/NumberTheory/Liouville/Basic.lean,Mathlib/NumberTheory/Liouville/LiouvilleNumber.lean,Mathlib/NumberTheory/Modular.lean,Mathlib/NumberTheory/ModularForms/EisensteinSeries/Defs.lean,Mathlib/NumberTheory/ModularForms/Identities.lean,Mathlib/NumberTheory/ModularForms/JacobiTheta/OneVariable.lean,Mathlib/NumberTheory/ModularForms/SlashActions.lean,Mathlib/NumberTheory/ModularForms/SlashInvariantForms.lean,Mathlib/NumberTheory/MulChar/Lemmas.lean,Mathlib/NumberTheory/NumberField/Basic.lean,Mathlib/NumberTheory/NumberField/CanonicalEmbedding/Basic.lean,Mathlib/NumberTheory/NumberField/ClassNumber.lean,Mathlib/NumberTheory/NumberField/Discriminant.lean,Mathlib/NumberTheory/NumberField/Embeddings.lean,Mathlib/NumberTheory/NumberField/FractionalIdeal.lean,Mathlib/NumberTheory/NumberField/Norm.lean,Mathlib/NumberTheory/NumberField/Units/DirichletTheorem.lean,Mathlib/RepresentationTheory/Maschke.lean,Mathlib/RingTheory/Adjoin/Basic.lean,Mathlib/RingTheory/Adjoin/FG.lean,Mathlib/RingTheory/AlgebraTower.lean,Mathlib/RingTheory/Discriminant.lean,Mathlib/RingTheory/FractionalIdeal/Norm.lean,Mathlib/RingTheory/Ideal/Norm.lean,Mathlib/RingTheory/IntegralClosure/IsIntegralClosure/Basic.lean,Mathlib/RingTheory/Localization/Basic.lean,Mathlib/RingTheory/Localization/FractionRing.lean,Mathlib/RingTheory/Polynomial/Cyclotomic/Eval.lean,Mathlib/RingTheory/Polynomial/Cyclotomic/Expand.lean,Mathlib/RingTheory/Polynomial/Cyclotomic/Roots.lean,Mathlib/RingTheory/Polynomial/GaussLemma.lean,Mathlib/RingTheory/Polynomial/Hermite/Gaussian.lean,Mathlib/RingTheory/Polynomial/Pochhammer.lean,Mathlib/RingTheory/RootsOfUnity/Lemmas.lean,Mathlib/RingTheory/RootsOfUnity/Minpoly.lean,Mathlib/RingTheory/TensorProduct/Basic.lean,Mathlib/RingTheory/Trace/Basic.lean,Mathlib/RingTheory/WittVector/Basic.lean,Mathlib/RingTheory/WittVector/Defs.lean,Mathlib/RingTheory/WittVector/Frobenius.lean,Mathlib/RingTheory/WittVector/InitTail.lean,Mathlib/RingTheory/WittVector/IsPoly.lean,Mathlib/RingTheory/WittVector/MulP.lean,Mathlib/RingTheory/WittVector/StructurePolynomial.lean,Mathlib/RingTheory/WittVector/Verschiebung.lean |
80 |
6 |
['eric-wieser', 'github-actions', 'leanprover-bot', 'mattrobball'] |
nobody |
133-11045 4 months ago |
133-11045 4 months ago |
0-0 0 seconds |
14803 |
StevenClontz author:StevenClontz |
chore: use `Disjoint` nhd filters for all separation axioms |
---
[](https://gitpod.io/from-referrer/)
|
t-topology
merge-conflict
|
157/122 |
Mathlib/Topology/Separation.lean |
1 |
1 |
['github-actions'] |
nobody |
133-11040 4 months ago |
133-11041 4 months ago |
0-0 0 seconds |
14675 |
adomani author:adomani |
dev: the repeated variable linter |
---
[](https://gitpod.io/from-referrer/)
|
t-linter
merge-conflict
WIP
|
71/0 |
Mathlib/Tactic/Linter/Lint.lean |
1 |
1 |
['github-actions'] |
nobody |
133-11035 4 months ago |
133-11035 4 months ago |
0-8 8 seconds |
14330 |
Ruben-VandeVelde author:Ruben-VandeVelde |
chore: split Mathlib.Algebra.Star.Basic |
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict
awaiting-author
|
446/331 |
Mathlib.lean,Mathlib/Algebra/Module/LinearMap/Star.lean,Mathlib/Algebra/Star/Basic.lean,Mathlib/Algebra/Star/BigOperators.lean,Mathlib/Algebra/Star/Defs.lean,Mathlib/Algebra/Star/Lemmas.lean,Mathlib/Algebra/Star/Order.lean,Mathlib/Algebra/Star/Pi.lean,Mathlib/Algebra/Star/Pointwise.lean,Mathlib/Algebra/Star/Rat.lean,Mathlib/Algebra/Star/Regular.lean,Mathlib/Algebra/Star/StarRingHom.lean,Mathlib/Analysis/NormedSpace/LinearIsometry.lean,Mathlib/Data/Complex/Basic.lean,scripts/noshake.json |
15 |
3 |
['github-actions', 'grunweg', 'j-loreaux'] |
nobody |
133-10995 4 months ago |
133-11021 4 months ago |
0-45204 12 hours |
14023 |
mattrobball author:mattrobball |
perf(RingTheory.OreLocalization): make data irreducible |
We generally do not want to unfold operations passing through `Quotient` if we can avoid it for performance reasons.
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict |
43/32 |
Mathlib/GroupTheory/MonoidLocalization.lean,Mathlib/RingTheory/OreLocalization/Basic.lean,Mathlib/RingTheory/OreLocalization/Ring.lean |
3 |
5 |
['github-actions', 'grunweg', 'leanprover-bot', 'mattrobball'] |
nobody |
133-10890 4 months ago |
441-713 1 year ago |
0-0 0 seconds |
14007 |
adomani author:adomani |
test: papercut linter working on all mathlib |
This PR is a testing ground for potential issues with the papercut linter #13999. It is not intended to be merged.
The linter is active on all of mathlib, to make sure that the linter does not throw errors, but only emits warnings!
---
[](https://gitpod.io/from-referrer/)
|
t-linter
merge-conflict
WIP
|
249/0 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter.lean,Mathlib/Tactic/Linter/Papercut.lean,test/Papercut.lean |
5 |
1 |
['github-actions'] |
nobody |
133-10880 4 months ago |
133-10880 4 months ago |
0-0 0 seconds |
20354 |
eric-wieser author:eric-wieser |
feat: generalize `ContinuousLinearMap.curry` to TVS |
Follow on from #10777
---
[](https://gitpod.io/from-referrer/)
|
t-analysis
merge-conflict
|
57/25 |
Mathlib/Analysis/NormedSpace/Multilinear/Curry.lean |
1 |
3 |
['eric-wieser', 'github-actions', 'leanprover-community-bot-assistant'] |
nobody |
133-10815 4 months ago |
133-10815 4 months ago |
0-0 0 seconds |
11523 |
thorimur author:thorimur |
bench: test syntax linter |
---
The purpose of this PR is just to bench the "best-case scenario" for a linter which iterates through syntax, updating and checking a simple counter along the way.
[](https://gitpod.io/from-referrer/)
|
t-linter
merge-conflict
|
22/0 |
Mathlib.lean,Mathlib/Command/Linter.lean,Mathlib/Tactic/Common.lean |
3 |
3 |
['grunweg', 'leanprover-bot', 'thorimur'] |
nobody |
133-10724 4 months ago |
133-10724 4 months ago |
0-0 0 seconds |
8511 |
eric-wieser author:eric-wieser |
refactor(MeasureTheory/Measure/Haar/Basic): partially generalize to the affine case |
Without a `Mul` version of `AddTorsor`, this generalization can only go so far.
---
[](https://gitpod.io/from-referrer/)
|
t-measure-probability
merge-conflict
awaiting-author
|
52/46 |
Mathlib/MeasureTheory/Measure/Haar/Basic.lean |
1 |
0 |
[] |
nobody |
133-10626 4 months ago |
133-10626 4 months ago |
0-0 0 seconds |
7994 |
ericrbg author:ericrbg |
chore: generalize `LieSubalgebra.mem_map_submodule` |
---
Not sure if we should rename to something like `mem_map_iff_mem_map_submodule` or not.
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
please-adopt
label:t-algebra$ |
16/4 |
Mathlib/Algebra/Lie/SkewAdjoint.lean,Mathlib/Algebra/Lie/Subalgebra.lean |
2 |
3 |
['eric-wieser', 'ericrbg'] |
nobody |
133-10614 4 months ago |
133-10614 4 months ago |
0-0 0 seconds |
6317 |
eric-wieser author:eric-wieser |
refactor(Data/Finsupp/Defs): make Finsupp.single defeq to Pi.single |
By adding a `DecidableEq ι` argument to `Finsupp.single`, we remove the reference to `Classical.decEq ι` in the definition, which in turn means that when coerced to a function it is now defeq to `Pi.single`.
This also brings it in line with `DFinsupp.single`.
This does not go as far as making `Finsupp.single` computable.
---
[](https://gitpod.io/from-referrer/)
|
t-data
merge-conflict
WIP
|
269/226 |
Mathlib/Algebra/BigOperators/Finsupp.lean,Mathlib/Data/Finsupp/AList.lean,Mathlib/Data/Finsupp/Basic.lean,Mathlib/Data/Finsupp/Defs.lean,Mathlib/Data/Finsupp/Fintype.lean,Mathlib/Data/Finsupp/Indicator.lean,Mathlib/Data/Finsupp/Multiset.lean,Mathlib/Data/Finsupp/Order.lean,Mathlib/Data/Finsupp/ToDFinsupp.lean,Mathlib/Data/Nat/Choose/Multinomial.lean,Mathlib/LinearAlgebra/Basis.lean,Mathlib/LinearAlgebra/Finsupp.lean |
12 |
0 |
[] |
nobody |
133-10608 4 months ago |
133-10608 4 months ago |
0-0 0 seconds |
6277 |
jjaassoonn author:jjaassoonn |
Dimension theory |
Some results are
- The ring Krull dimension and the topological dimension of the prime spectrum of a ring are the same
- A field is zero-dimensional and a PID that is not a field is one dimensional
- An Artinian ring is zero-dimensional
- The Krull dimension of ring $R$ is equal to the supremum of heights of maximal ideals [00KG](https://stacks.math.columbia.edu/tag/00KG)
- two definitions of module length agree
- A module is finite length iff both artinian and noetherian
- length of module $M$ is equal to the sum of length of $N$ and length of $M / N$ where $N$ is a submodule of $M$.
- Noetherian ring has only finitely many minimal primes #9088
- In a zero dimensional ring, prime ideals are maximal
- Artinian rings has finitely many maximal ideals #9087
- zero-dimensional rings with finitely many prime ideals are products of its localizations: $R \cong \prod_{\mathfrak{p}}R_{\mathfrak{p}}$
- Let $M_0 \le ... \le M_n$, then $l(M_n/ M_0) = l(M_1/M_0) + l(M_2/M_1) + ... + l(M_n/M_{n-1})$ where $l$ denotes module length.
- If $f : R \to S$ is a ring homomorphism and $M$ an $S$-module, then $l_R(M) \le l_S(M)$, when $f$ is surjective then they are equal. (Note that this is expressed using `[Algebra R S]` and `RestrictScalars R S M`, instead of a literal ring hom)
- Artinian rings are noetherian ring of dimension 0.
- For 0-dimensional local ring, its maximal ideal is locally nilpotent
- In notherian ring, $I \le \sqrt{J}$ implies $I ^ n \le J$ for some $n$
---
- [x] depends on: #6309
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
label:t-algebra$ |
3289/459 |
Mathlib.lean,Mathlib/Algebra/Module/Length.lean,Mathlib/Algebra/Module/Submodule/JordanHolder.lean,Mathlib/Algebra/PUnitInstances.lean,Mathlib/AlgebraicGeometry/PrimeSpectrum/ArtinianAndNoetherian.lean,Mathlib/Data/List/Basic.lean,Mathlib/Data/List/Dedup.lean,Mathlib/Data/List/Nodup.lean,Mathlib/LinearAlgebra/Quotient.lean,Mathlib/Order/Cover.lean,Mathlib/Order/JordanHolder.lean,Mathlib/Order/KrullDimension.lean,Mathlib/Order/ListOnPartialOrderTypes.lean,Mathlib/Order/Monotone/Basic.lean,Mathlib/Order/RelSeries.lean,Mathlib/RingTheory/Artinian.lean,Mathlib/RingTheory/Finiteness.lean,Mathlib/RingTheory/Ideal/Operations.lean,Mathlib/RingTheory/Ideal/Pi.lean,Mathlib/RingTheory/KrullDimension.lean,Mathlib/RingTheory/Noetherian.lean,Mathlib/RingTheory/SimpleModule.lean,Mathlib/Topology/KrullDimension.lean,Mathlib/Topology/Sheaves/SheafCondition/EqualizerProducts.lean |
24 |
11 |
['alreadydone', 'jjaassoonn', 'leanprover-community-mathlib4-bot'] |
nobody |
133-10603 4 months ago |
564-67016 1 year ago* |
0-0 0 seconds* |
4979 |
mhk119 author:mhk119 |
doc(Data/Nat/Bitblast): initial commit |
Initial commit of Bitblast.lean where we prove equivalence of bitblast unsigned less than and bitblast addition.
---
[](https://gitpod.io/from-referrer/)
|
t-data
merge-conflict
|
202/4 |
Mathlib/Data/Bool/Basic.lean,Mathlib/Data/Nat/Bitwise.lean,Mathlib/Data/Nat/Pow.lean |
3 |
49 |
['ChrisHughes24', 'digama0', 'goens', 'grunweg', 'j-loreaux', 'kim-em', 'mhk119'] |
nobody |
133-10592 4 months ago |
133-10592 4 months ago |
7-68358 7 days |
8536 |
jjaassoonn author:jjaassoonn |
characteristic predicate of tensor product |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
label:t-algebra$ |
399/7 |
Mathlib/Algebra/Category/AlgebraCat/Monoidal.lean,Mathlib/LinearAlgebra/IsTensorProduct.lean,Mathlib/LinearAlgebra/TensorProduct.lean,Mathlib/LinearAlgebra/TensorProduct/Tower.lean |
4 |
12 |
['alreadydone', 'eric-wieser', 'jjaassoonn'] |
nobody |
133-10556 4 months ago |
133-10556 4 months ago |
0-0 0 seconds |
11524 |
mcdoll author:mcdoll |
refactor: Introduce type-class for SchwartzMap |
---
There are a lot of other refactors to do (`seminormAux` should have a nicer name and gobble up more theorems from `seminorm`), then one can prove `integrable` and friends with only `SchwartzMapClass`.
[](https://gitpod.io/from-referrer/)
|
t-analysis
merge-conflict
WIP
|
139/137 |
Mathlib/Analysis/Distribution/SchwartzSpace.lean,Mathlib/Analysis/Fourier/PoissonSummation.lean,Mathlib/Topology/ContinuousFunction/ZeroAtInfty.lean |
3 |
0 |
[] |
nobody |
133-10522 4 months ago |
133-10522 4 months ago |
0-0 0 seconds |
9819 |
jjaassoonn author:jjaassoonn |
fg graded ring |
1. if $A$ is a noetherian graded ring, then $A_0$ is a noetherian subring of $A$ and $A$ is a finitely generated algebra over $A_0$, if $M$ is a finitely generated graded module over $A$, then each $M_n$ is a finitely generated module over
$A_0$.
2. Definition of additive functions over any abelian category: if $C$ is an abelian category, a function $f : C \to \mathbb Z$ is said to be additive, if $f(y) = f(x) + f(z)$ whenever $0\to x \to y \to z \to 0$ is exact. proved some basic properties such as $f(0) = 0$ and $f(x) = f(y)$ whenever $x \cong y$ and interaction of $f$ with longer exact sequences
3. The category of finitely generated module over noetherian ring is abelian
4. A proof of Hilbert-Serre theorem: the Poincare series is actually of the form $\frac{p}{\prod(1- X^i)}$ where $p$ is polynomial
The code works, but poorly written.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
WIP
label:t-algebra$ |
6745/217 |
Mathlib.lean,Mathlib/Algebra/Category/FGModuleCat/Abelian.lean,Mathlib/Algebra/Category/FGModuleCat/Basic.lean,Mathlib/Algebra/Category/FGModuleCat/EpiMono.lean,Mathlib/Algebra/Category/FGModuleCat/Kernels.lean,Mathlib/Algebra/Category/FGModuleCat/Limits.lean,Mathlib/Algebra/DirectSum/Basic.lean,Mathlib/Algebra/GradedMonoid.lean,Mathlib/Algebra/HilbertSerre/AdditiveFunction.lean,Mathlib/Algebra/HilbertSerre/FiniteInstances.lean,Mathlib/Algebra/HilbertSerre/HilbertPolynomial.lean,Mathlib/Algebra/HilbertSerre/Theorem.lean,Mathlib/Algebra/Module/GradeZeroModule.lean,Mathlib/Algebra/Module/GradedModule.lean,Mathlib/AlgebraicGeometry/ProjectiveSpectrum/Topology.lean,Mathlib/RingTheory/FiniteType.lean,Mathlib/RingTheory/Finiteness.lean,Mathlib/RingTheory/GradedAlgebra/Basic.lean,Mathlib/RingTheory/GradedAlgebra/HomogeneousIdeal.lean,Mathlib/RingTheory/GradedAlgebra/Noetherian.lean,Mathlib/RingTheory/GradedAlgebra/Radical.lean,Mathlib/RingTheory/GradedAlgebra/Subgrading.lean,Mathlib/RingTheory/Polynomial/Hilbert.lean,Mathlib/RingTheory/PowerSeries/Basic.lean,Mathlib/RingTheory/PowerSeries/WellKnown.lean |
25 |
n/a |
['FMLJohn', 'github-actions'] |
nobody |
133-10504 4 months ago |
unknown |
unknown |
13543 |
adomani author:adomani |
test: automatically undeprecate |
A test for `update_deprecations`. There are two files with deprecated declarations, but CI automatically fixes them, so that they pass the noisy tests (as well as passing fail-on-warning `lake build`).
---
[](https://gitpod.io/from-referrer/)
|
t-linter
merge-conflict
|
345/4 |
.github/workflows/bors.yml,.github/workflows/build.yml,.github/workflows/build.yml.in,.github/workflows/build_fork.yml,Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/UpdateDeprecations.lean,Mathlib/test_depr.lean,Mathlib/test_depr_no_change.lean,lakefile.lean,scripts/update_deprecations.lean,test/UpdateDeprecations.lean |
12 |
0 |
[] |
nobody |
133-10355 4 months ago |
133-10355 4 months ago |
0-0 0 seconds |
14932 |
eric-wieser author:eric-wieser |
chore: add nndist versions of lemmas |
---
[](https://gitpod.io/from-referrer/)
|
t-analysis
merge-conflict
|
108/1 |
Mathlib/Analysis/InnerProductSpace/Basic.lean,Mathlib/Geometry/Euclidean/Basic.lean |
2 |
1 |
['github-actions'] |
nobody |
133-10168 4 months ago |
133-10168 4 months ago |
0-0 0 seconds |
22269 |
Thmoas-Guan author:Thmoas-Guan |
chore(Algebra): replace Submodule.quotient.mk with Submodule.mkQ |
Replace Submodule.quotient.mk with Submodule.mkQ as much as possible as it have better composition property and more direct lemmas, making it more similarly with `Ideal.Quotient.mk`
(except Algebra.Lie.Quotient.Basic for ones more familiar with these area)
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
awaiting-author
label:t-algebra$ |
431/218 |
Mathlib/Algebra/Exact.lean,Mathlib/Algebra/Module/CharacterModule.lean,Mathlib/Algebra/Module/LocalizedModule/Submodule.lean,Mathlib/Algebra/Module/PID.lean,Mathlib/Algebra/Module/Torsion.lean,Mathlib/Algebra/Module/ZLattice/Basic.lean,Mathlib/LinearAlgebra/Dimension/Constructions.lean,Mathlib/LinearAlgebra/Dimension/RankNullity.lean,Mathlib/LinearAlgebra/Dual/Lemmas.lean,Mathlib/LinearAlgebra/Isomorphisms.lean,Mathlib/LinearAlgebra/Projection.lean,Mathlib/LinearAlgebra/Quotient/Basic.lean,Mathlib/LinearAlgebra/Quotient/Defs.lean,Mathlib/LinearAlgebra/Quotient/Pi.lean,Mathlib/LinearAlgebra/SModEq.lean,Mathlib/LinearAlgebra/Semisimple.lean,Mathlib/LinearAlgebra/TensorProduct/Quotient.lean,Mathlib/LinearAlgebra/TensorProduct/RightExactness.lean,Mathlib/NumberTheory/RamificationInertia/Basic.lean,Mathlib/RepresentationTheory/GroupCohomology/LowDegree.lean,Mathlib/RingTheory/AdicCompletion/Algebra.lean,Mathlib/RingTheory/AdicCompletion/Basic.lean,Mathlib/RingTheory/AdicCompletion/Exactness.lean,Mathlib/RingTheory/AdicCompletion/Functoriality.lean,Mathlib/RingTheory/Flat/FaithfullyFlat/Basic.lean,Mathlib/RingTheory/Ideal/Colon.lean,Mathlib/RingTheory/Ideal/Quotient/Basic.lean,Mathlib/RingTheory/Ideal/Quotient/Defs.lean,Mathlib/RingTheory/Ideal/Quotient/Operations.lean,Mathlib/RingTheory/PowerBasis.lean,Mathlib/RingTheory/QuotSMulTop.lean,Mathlib/RingTheory/Smooth/Basic.lean,Mathlib/RingTheory/TensorProduct/Quotient.lean |
33 |
10 |
['Thmoas-Guan', 'alreadydone', 'erdOne', 'github-actions', 'grunweg', 'leanprover-bot'] |
nobody |
132-2907 4 months ago |
132-2907 4 months ago |
16-61571 16 days |
18202 |
ADedecker author:ADedecker |
chore: refactor algebraic filter bases |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-topology
merge-conflict
label:t-algebra$ |
1086/1315 |
Mathlib/Analysis/Distribution/SchwartzSpace.lean,Mathlib/Analysis/LocallyConvex/AbsConvex.lean,Mathlib/Analysis/LocallyConvex/Barrelled.lean,Mathlib/Analysis/LocallyConvex/WeakDual.lean,Mathlib/Analysis/LocallyConvex/WithSeminorms.lean,Mathlib/Analysis/Normed/Operator/WeakOperatorTopology.lean,Mathlib/FieldTheory/KrullTopology.lean,Mathlib/RingTheory/DedekindDomain/FiniteAdeleRing.lean,Mathlib/Topology/Algebra/FilterBasis.lean,Mathlib/Topology/Algebra/Module/UniformConvergence.lean,Mathlib/Topology/Algebra/Nonarchimedean/AdicTopology.lean,Mathlib/Topology/Algebra/Nonarchimedean/Bases.lean,Mathlib/Topology/Algebra/UniformFilterBasis.lean,Mathlib/Topology/Algebra/Valued/ValuationTopology.lean |
14 |
1 |
['github-actions'] |
nobody |
132-2839 4 months ago |
132-2839 4 months ago |
0-0 0 seconds |
23546 |
JovanGerb author:JovanGerb |
feat(LinearAlgebra/AffineSpace/AffineSubspace): rename `AffineSubspace.mk'` to `Submodule.shift` |
In addition to renaming, I've refactored the code a bit:
- `mem_mk'_iff_vsub_mem` was obsolete since it was the same as `mem_mk'`, so I removed it (this is due to a change in the definition I made recently)
- I added a nonempty instance for `shift`
- I added a simp lemma that `shift` isn't equal to `⊥` (the empty affine subspace). I need this for the next point.
- Edit: I'll leave this for a later PR.
~I proved a simp lemma that a `shift` is parallel to a `shift` if and only if the linear subspaces are the same.~
- I renamed `mk'_eq` to `shift_direction_eq_self `.
- I renamed `eq_or_eq_secondInter_of_mem_mk'_span_singleton_iff_mem` to `eq_or_eq_secondInter_iff_mem_of_mem_shift_span_singleton`. I think it is better to put the `of_mem_mk'_span_singleton` at the end of the name.
---
[](https://gitpod.io/from-referrer/)
|
t-euclidean-geometry
merge-conflict
|
128/99 |
Mathlib/Algebra/Module/ZLattice/Basic.lean,Mathlib/Geometry/Euclidean/Basic.lean,Mathlib/Geometry/Euclidean/MongePoint.lean,Mathlib/Geometry/Euclidean/PerpBisector.lean,Mathlib/Geometry/Euclidean/Sphere/SecondInter.lean,Mathlib/Geometry/Euclidean/Sphere/Tangent.lean,Mathlib/LinearAlgebra/AffineSpace/AffineSubspace/Defs.lean |
7 |
4 |
['JovanGerb', 'github-actions', 'leanprover-community-bot-assistant'] |
nobody |
131-71739 4 months ago |
131-71740 4 months ago |
26-25420 26 days |
19315 |
quangvdao author:quangvdao |
feat(Data/Finsupp/Fin): Add `Finsupp` operations on `Fin` tuple |
This PR adds more analogues of operations on `Fin` tuples to the `Finsupp` setting. Before, there were only `Finsupp.cons` and `Finsupp.tail`. Now there are also `Finsupp.snoc`, `Finsupp.insertNth`, `Finsupp.init`, and `Finsupp.removeNth`. These all come with supporting lemmas.
I also removed the porting comment about `succAboveCases` in `Data/Fin/Basic`, and added a lemma about `succAbove` in `Data/Fin/Tuple/Basic`.
---
- [x] depends on: #20361
- [x] depends on: #20771
- [x] depends on: #20770
[](https://gitpod.io/from-referrer/)
|
t-data
merge-conflict
awaiting-author
|
193/16 |
Mathlib/Algebra/BigOperators/Fin.lean,Mathlib/Algebra/BigOperators/Finsupp.lean,Mathlib/Algebra/MvPolynomial/Equiv.lean,Mathlib/Data/Finsupp/Fin.lean,Mathlib/RingTheory/MvPolynomial/Homogeneous.lean,scripts/nolints_prime_decls.txt |
6 |
44 |
['YaelDillies', 'github-actions', 'j-loreaux', 'kbuzzard', 'mathlib4-dependent-issues-bot', 'quangvdao'] |
nobody |
129-45998 4 months ago |
129-45998 4 months ago |
43-81255 43 days |
19464 |
adomani author:adomani |
test: removed merge-conflict |
---
[](https://gitpod.io/from-referrer/)
|
CI
merge-conflict
delegated
WIP
|
22/1 |
.github/workflows/PR_summary.yml,scripts/zulip_emoji_merge_delegate.py |
2 |
10 |
['adomani', 'github-actions', 'leanprover-community-bot-assistant'] |
nobody |
128-57322 4 months ago |
128-57324 4 months ago |
0-0 0 seconds |
7907 |
urkud author:urkud |
feat: introduce `NthRoot` notation class |
Also use it for `Real.sqrt`, and replace the few occurrences of `sqrt` that do not already use the notation.
---
[Zulip](https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/.60Sqrt.60.20notation.20typeclass/near/400086502)
[](https://gitpod.io/from-referrer/) |
t-algebra
t-analysis
awaiting-CI
merge-conflict
label:t-algebra$ |
193/156 |
Archive/Imo/Imo1959Q2.lean,Archive/Imo/Imo1960Q2.lean,Archive/Imo/Imo2001Q2.lean,Archive/Imo/Imo2006Q3.lean,Archive/Imo/Imo2008Q3.lean,Archive/Imo/Imo2008Q4.lean,Archive/Sensitivity.lean,Archive/Wiedijk100Theorems/AreaOfACircle.lean,Mathlib.lean,Mathlib/Algebra/NthRoot.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Instances.lean,Mathlib/Analysis/Complex/AbelLimit.lean,Mathlib/Analysis/RCLike/Basic.lean,Mathlib/Analysis/SpecialFunctions/Pow/Asymptotics.lean,Mathlib/Analysis/SpecialFunctions/Pow/Real.lean,Mathlib/Analysis/SpecialFunctions/Stirling.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Basic.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Bounds.lean,Mathlib/Data/Real/GoldenRatio.lean,Mathlib/Data/Real/Sqrt.lean,Mathlib/LinearAlgebra/Matrix/PosDef.lean,Mathlib/MeasureTheory/Measure/Lebesgue/VolumeOfBalls.lean,Mathlib/NumberTheory/Harmonic/GammaDeriv.lean,Mathlib/NumberTheory/NumberField/CanonicalEmbedding/ConvexBody.lean,Mathlib/NumberTheory/NumberField/ClassNumber.lean,Mathlib/NumberTheory/NumberField/Discriminant/Basic.lean,Mathlib/Probability/Distributions/Gaussian.lean,MathlibTest/positivity.lean |
28 |
9 |
['eric-wieser', 'github-actions', 'kmill', 'urkud'] |
nobody |
127-73112 4 months ago |
382-270 1 year ago |
0-0 0 seconds |
9273 |
grunweg author:grunweg |
feat: extended charts are local diffeomorphisms on their source |
---
TODO: I think this should hold at any interior point - as the inverse of the extended chart, restricted to the interior of its source, will be a local inverse.
The analogous result for un-extended charts is shown in #8160.
Unresolved questions
- are all the tiny API lemmas useful; are any more missing?
- do I want similar results for `extChartAt`? (In any case, they are easy to deduce.)
- [ ] depends on: #8738 for simplicity
[](https://gitpod.io/from-referrer/)
|
t-differential-geometry
merge-conflict
|
225/12 |
Mathlib/Geometry/Manifold/ContMDiff/Atlas.lean,Mathlib/Geometry/Manifold/LocalDiffeomorph.lean,Mathlib/Topology/Algebra/Module/Basic.lean |
3 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
127-47147 4 months ago |
unknown |
unknown |
24248 |
urkud author:urkud |
feat(HaarToSphere): add integrability lemmas |
---
[](https://gitpod.io/from-referrer/)
|
t-measure-probability
merge-conflict
|
99/6 |
Mathlib/MeasureTheory/Constructions/HaarToSphere.lean,Mathlib/MeasureTheory/Integral/Prod.lean |
2 |
2 |
['github-actions', 'leanprover-community-bot-assistant'] |
nobody |
125-11177 4 months ago |
125-11179 4 months ago |
0-0 0 seconds |
24019 |
urkud author:urkud |
feat(Analysis): Poincaré lemma for 1-forms |
---
[](https://gitpod.io/from-referrer/)
|
t-analysis
merge-conflict
|
704/33 |
Mathlib.lean,Mathlib/Analysis/Calculus/ContDiff/Basic.lean,Mathlib/Analysis/Calculus/Deriv/Basic.lean,Mathlib/Analysis/Calculus/Deriv/CompMul.lean,Mathlib/Analysis/Calculus/Deriv/Shift.lean,Mathlib/Analysis/Calculus/FDeriv/Analytic.lean,Mathlib/Analysis/Calculus/FDeriv/Basic.lean,Mathlib/Analysis/Calculus/FDeriv/Equiv.lean,Mathlib/Analysis/Calculus/Gradient/Basic.lean,Mathlib/Analysis/Calculus/Poincare/OneForm.lean,Mathlib/Analysis/Calculus/TangentCone.lean,Mathlib/MeasureTheory/Integral/DivergenceTheorem.lean,Mathlib/MeasureTheory/Integral/PathIntegral/Basic.lean,Mathlib/Topology/Homotopy/Path.lean,Mathlib/Topology/Path.lean,Mathlib/Topology/UnitInterval.lean |
16 |
4 |
['github-actions', 'leanprover-community-bot-assistant'] |
nobody |
124-56686 4 months ago |
124-56688 4 months ago |
0-0 0 seconds |
24642 |
grunweg author:grunweg |
WIP-feat: add layercake formula for ENNReal-valued functions |
Not much to see here yet; some significant amount of work remains.
---
- [ ] depends on: #24643
- [ ] depends on: #24640 (based on that PR for simplicity)
[](https://gitpod.io/from-referrer/)
|
carleson
t-analysis
merge-conflict
WIP
|
189/24 |
Mathlib/Analysis/SpecialFunctions/Pow/Integral.lean,Mathlib/MeasureTheory/Function/LpSeminorm/Basic.lean,Mathlib/MeasureTheory/Function/LpSpace/Basic.lean,Mathlib/MeasureTheory/Integral/Layercake.lean |
4 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
123-65997 4 months ago |
123-66000 4 months ago |
0-0 0 seconds |
21712 |
grunweg author:grunweg |
chore: generalise more lemmas to `ContinuousENorm` |
---
- [x] depends on: #21781 (minor drive-by clean-up)
- [x] depends on: #21670
- [x] depends on: #22708 (extracted from this)
- some parts depend on #21433 (or better: #22175); when the dependent PR has landed, I will re-assess whether to split these into a separate PR
[](https://gitpod.io/from-referrer/)
|
carleson
t-measure-probability
awaiting-CI
merge-conflict
|
76/31 |
Mathlib/Analysis/Normed/MulAction.lean,Mathlib/MeasureTheory/Function/LpSeminorm/Basic.lean,Mathlib/MeasureTheory/Function/LpSpace/Basic.lean,Mathlib/MeasureTheory/Function/LpSpace/ContinuousFunctions.lean |
4 |
5 |
['github-actions', 'grunweg', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
123-1281 4 months ago |
133-11315 4 months ago |
0-0 0 seconds |
21375 |
grunweg author:grunweg |
WIP: generalise lemmas to ENorm |
This work is part of (and a necessary pre-requisite for) the Carleson project.
---
[](https://gitpod.io/from-referrer/)
|
carleson
t-measure-probability
awaiting-CI
merge-conflict
WIP
|
471/221 |
Mathlib/Analysis/NormedSpace/IndicatorFunction.lean,Mathlib/MeasureTheory/Function/L2Space.lean,Mathlib/MeasureTheory/Function/LocallyIntegrable.lean,Mathlib/MeasureTheory/Function/LpOrder.lean,Mathlib/MeasureTheory/Function/LpSeminorm/Basic.lean,Mathlib/MeasureTheory/Function/LpSeminorm/ChebyshevMarkov.lean,Mathlib/MeasureTheory/Function/LpSeminorm/CompareExp.lean,Mathlib/MeasureTheory/Function/LpSeminorm/TriangleInequality.lean,Mathlib/MeasureTheory/Function/LpSeminorm/Trim.lean,Mathlib/MeasureTheory/Function/LpSpace.lean,Mathlib/MeasureTheory/Function/SimpleFuncDenseLp.lean,Mathlib/MeasureTheory/Function/UniformIntegrable.lean,Mathlib/Probability/Independence/Integrable.lean |
13 |
2 |
['fpvandoorn', 'grunweg'] |
nobody |
122-82056 3 months ago |
133-11310 4 months ago |
0-0 0 seconds |
24378 |
urkud author:urkud |
feat(Algebra/Order/Field/Basic): generalize lemmas |
... from linear ordered semifields to (commutative) groups with zero.
---
I'm going to do another round of generalizing today or tomorrow, so making it a draft PR for now.
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
label:t-algebra$ |
183/181 |
Archive/OxfordInvariants/Summer2021/Week3P1.lean,Mathlib/Algebra/Order/Field/Basic.lean,Mathlib/Algebra/Order/Floor/Ring.lean,Mathlib/Algebra/Order/Floor/Semiring.lean,Mathlib/Algebra/Order/GroupWithZero/Unbundled/Basic.lean,Mathlib/Analysis/Analytic/Basic.lean,Mathlib/Analysis/Asymptotics/Lemmas.lean,Mathlib/Analysis/CStarAlgebra/ApproximateUnit.lean,Mathlib/Analysis/Calculus/BumpFunction/Basic.lean,Mathlib/Analysis/Calculus/BumpFunction/FiniteDimension.lean,Mathlib/Analysis/Calculus/BumpFunction/InnerProduct.lean,Mathlib/Analysis/Complex/AbelLimit.lean,Mathlib/Analysis/Complex/Hadamard.lean,Mathlib/Analysis/Convex/Segment.lean,Mathlib/Analysis/Convex/SpecificFunctions/Basic.lean,Mathlib/Analysis/Convex/SpecificFunctions/Pow.lean,Mathlib/Analysis/Convex/StrictConvexSpace.lean,Mathlib/Analysis/Convex/Uniform.lean,Mathlib/Analysis/Convex/Visible.lean,Mathlib/Analysis/Fourier/RiemannLebesgueLemma.lean,Mathlib/Analysis/FunctionalSpaces/SobolevInequality.lean,Mathlib/Analysis/MeanInequalitiesPow.lean,Mathlib/Analysis/Normed/Field/Lemmas.lean,Mathlib/Analysis/Normed/Field/Ultra.lean,Mathlib/Analysis/Normed/Unbundled/SmoothingSeminorm.lean,Mathlib/Analysis/NormedSpace/HomeomorphBall.lean,Mathlib/Analysis/NormedSpace/OperatorNorm/NormedSpace.lean,Mathlib/Analysis/NormedSpace/Pointwise.lean,Mathlib/Analysis/SpecialFunctions/Complex/Arg.lean,Mathlib/Analysis/SpecialFunctions/Gamma/Beta.lean,Mathlib/Analysis/SpecialFunctions/Log/Deriv.lean,Mathlib/Analysis/SpecialFunctions/MulExpNegMulSqIntegral.lean,Mathlib/Analysis/SpecialFunctions/SmoothTransition.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Bounds.lean,Mathlib/Analysis/SpecificLimits/Basic.lean,Mathlib/Analysis/SpecificLimits/FloorPow.lean,Mathlib/Analysis/SpecificLimits/Normed.lean,Mathlib/Combinatorics/Additive/AP/Three/Behrend.lean,Mathlib/Combinatorics/Schnirelmann.lean,Mathlib/Combinatorics/SimpleGraph/Regularity/Chunk.lean,Mathlib/Computability/AkraBazzi/AkraBazzi.lean,Mathlib/Computability/AkraBazzi/GrowsPolynomially.lean,Mathlib/Data/Nat/Cast/Order/Field.lean,Mathlib/Data/Real/Archimedean.lean,Mathlib/Data/Real/Cardinality.lean,Mathlib/Data/Real/Pi/Wallis.lean,Mathlib/Geometry/Euclidean/Angle/Unoriented/Affine.lean,Mathlib/Geometry/Euclidean/Angle/Unoriented/RightAngle.lean,Mathlib/Geometry/Euclidean/Sphere/Tangent.lean,Mathlib/MeasureTheory/Function/StronglyMeasurable/Basic.lean,Mathlib/MeasureTheory/Function/UniformIntegrable.lean,Mathlib/MeasureTheory/Integral/CircleIntegral.lean,Mathlib/MeasureTheory/Integral/MeanInequalities.lean,Mathlib/MeasureTheory/Integral/PeakFunction.lean,Mathlib/MeasureTheory/Measure/SeparableMeasure.lean,Mathlib/NumberTheory/Bertrand.lean,Mathlib/NumberTheory/ClassNumber/AdmissibleAbs.lean,Mathlib/NumberTheory/DiophantineApproximation/Basic.lean,Mathlib/NumberTheory/LSeries/Injectivity.lean,Mathlib/NumberTheory/LSeries/ZMod.lean,Mathlib/NumberTheory/NumberField/Discriminant/Basic.lean,Mathlib/NumberTheory/Padics/Hensel.lean,Mathlib/NumberTheory/Padics/MahlerBasis.lean,Mathlib/NumberTheory/Pell.lean,Mathlib/NumberTheory/Transcendental/Liouville/LiouvilleNumber.lean,Mathlib/Order/Filter/AtTopBot/Floor.lean,Mathlib/Order/Interval/Set/IsoIoo.lean,Mathlib/Probability/StrongLaw.lean,Mathlib/RingTheory/Perfection.lean,Mathlib/Topology/ContinuousMap/Polynomial.lean,Mathlib/Topology/Instances/AddCircle.lean,Mathlib/Topology/UrysohnsLemma.lean |
72 |
3 |
['github-actions', 'leanprover-community-bot-assistant'] |
nobody |
122-66386 3 months ago |
122-66388 3 months ago |
0-0 0 seconds |
13685 |
niklasmohrin author:niklasmohrin |
feat(Combinatorics): add definitions for network flows |
Although we might not have any super-interesting results ready for mathlib yet, I feel that the definitions from this commit are already mature enough to include.
These definitions are ported from last semester's work we did at https://github.com/niklasmohrin/lean-seminar-2023 and I have put some time in to refactor our code to `Int` and now to any parameter `R`. In the linked repository, there is some more stuff that I can send in.
One obstacle without integer values is that it is not clear why a maximum flow would exist. I think the best way to tackle this would be to prove max-flow-min-cut theorem and implement the Ford-Fulkerson algorithm. It has been pointed out on Zulip that there is an [Isabelle formalization of the Edmonds Karp Algorithm](https://www.isa-afp.org/entries/EdmondsKarp_Maxflow.html).
I feel that the definitions are pretty solid and it makes sense to include them, even if just for unifying definitions across downstream projects.
---
[](https://gitpod.io/from-referrer/) |
new-contributor
t-combinatorics
merge-conflict
awaiting-author
|
244/0 |
Mathlib.lean,Mathlib/Combinatorics/Flow/Basic.lean,docs/references.bib |
3 |
57 |
['Shreyas4991', 'YaelDillies', 'b-mehta', 'github-actions', 'leanprover-community-bot-assistant', 'madvorak', 'niklasmohrin'] |
nobody |
121-36235 3 months ago |
121-36237 3 months ago |
86-21072 86 days |
15115 |
kkytola author:kkytola |
feat: Generalize assumptions in liminf and limsup results in ENNReals |
In a [review comment](https://github.com/leanprover-community/mathlib4/pull/13938#discussion_r1649744441) it was pointed out that results about liminf and limsup in ENNReal hold under milder assumptions. This PR does the generalization.
---
This PR is split off from #13938, where the review comment was made. The changes needed for the suggested generalization were of different kind than the simple PR's content, justifying a separate PR.
- [x] depends on: #13938
[](https://gitpod.io/from-referrer/)
|
t-order
t-topology
merge-conflict
awaiting-author
help-wanted
|
215/27 |
Mathlib/MeasureTheory/Measure/Portmanteau.lean,Mathlib/Order/LiminfLimsup.lean,Mathlib/Topology/Instances/ENNReal.lean |
3 |
8 |
['Ruben-VandeVelde', 'github-actions', 'grunweg', 'j-loreaux', 'kkytola', 'leanprover-community-mathlib4-bot'] |
nobody |
120-78391 3 months ago |
145-62695 4 months ago |
21-25493 21 days |
17129 |
joneugster author:joneugster |
feat(Tactic/Linter): add unicode linter for unicode variant-selectors |
Unicode characters can be followed by one of the two "variant-selectors" `\FE0E` (text) or `\FE0F` (emoji).
These appear to the user as a single unicode character and they might copy them by accident. For example `✅️` (`\u2705\uFE0F`), `✅` (`\u2705`) and `✅︎` (`\u2705\uFE0E`) are three variants of the "same" unicode character. The one without variant-selector might display as either emoji or not, depending on the user's device and font.
Add unicode linter ensuring variant-selector only appear on specified characters and also ensuring these characters always have the correct variant selector to avoid confusions.
Everything flagged by this linter can be fixed fully automatically with `lake exe lint-style --fix` or by commenting `bot fix style` on the PR.
---
- tracking PR: #16215
## Zulip discussions:
- https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/Whitelist.20for.20Unicode.3F
- https://leanprover.zulipchat.com/#narrow/stream/113488-general/topic/Lean.20specific.20font
## Related PRs:
- leanprover/lean4#5015 added some emoji-variant selectors to Emojis used in `Lean` itself.
[](https://gitpod.io/from-referrer/)
|
large-import
t-linter
merge-conflict
delegated
awaiting-author
|
245/14 |
Mathlib.lean,Mathlib/GroupTheory/GroupExtension/Defs.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter/TextBased.lean,Mathlib/Tactic/Linter/UnicodeLinter.lean,Mathlib/Tactic/Widget/Calc.lean,Mathlib/Tactic/Widget/CongrM.lean,Mathlib/Tactic/Widget/Conv.lean,Mathlib/Tactic/Widget/GCongr.lean,Mathlib/Topology/ContinuousMap/Weierstrass.lean,MathlibTest/LintStyleTextBased.lean |
11 |
25 |
['YaelDillies', 'adomani', 'github-actions', 'grunweg', 'joneugster', 'kim-em', 'leanprover-community-bot-assistant'] |
nobody |
119-66897 3 months ago |
119-66899 3 months ago |
82-54712 82 days |
17131 |
joneugster author:joneugster |
feat(Tactic/Linter): add unicode linter for unwanted characters |
Add unicode linter flagging bad unicode characters. In this first form, the linter only flags `\u00A0` (non-breaking space) and replaces it with a normal space. Non-breaking space has been chosen because they keep reappearing in mathlib and it seems to be uncontroversial to lint for these.
The whitelist/blacklist could then be refined in future PRs.
Everything flagged by this linter can be fixed fully automatically with `lake exe lint-style --fix` or by commenting `bot fix style` on the PR.
---
- tracking PR: #16215
## Zulip discussions:
- https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/Whitelist.20for.20Unicode.3F
- https://leanprover.zulipchat.com/#narrow/stream/113488-general/topic/Lean.20specific.20font
[](https://gitpod.io/from-referrer/)
|
large-import
t-linter
merge-conflict
awaiting-author
|
112/8 |
Mathlib.lean,Mathlib/Algebra/Lie/Semisimple/Lemmas.lean,Mathlib/Analysis/Analytic/IsolatedZeros.lean,Mathlib/CategoryTheory/Category/ReflQuiv.lean,Mathlib/LinearAlgebra/Vandermonde.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter/TextBased.lean,Mathlib/Tactic/Linter/UnicodeLinter.lean |
8 |
6 |
['github-actions', 'grunweg', 'leanprover-community-bot-assistant'] |
adomani and grunweg assignee:grunweg assignee:adomani |
119-66896 3 months ago |
119-66898 3 months ago |
52-18594 52 days |
8495 |
jjaassoonn author:jjaassoonn |
feat : Tensor-Hom adjunction in the category of modules |
# Tensor-Hom adjunction
Let $R$ be a commutative ring and $S$ any ring. Let $X$ be an $(S,R)$-bimoule. Then the tensor functor $(X \otimes_R \cdot)$ is a functor from left $R$-modules to left $S$-modules; and the hom-functor $Hom_S(X, \cdot)$ is a functor from left $S$-modules to left $R$-modules. For another left $S$-module $Y$, the left $R$-module structure of $Hom_S(X, Y)$ is given by $s \cdot f := x \mapsto f(s \cdot x)$. These two functors are adjoint.. In particular we have that
```math
{\rm Hom}_{S}(X\otimes_R Y, Z) \cong {\rm Hom}_R (Y, {\rm Hom}_S (X, Z))
```
## Implementation notes
1. Why not use the `Mathlib/LinearAlgebra/TensorProduct/Tower.lean`
In our setting `X` is an `(R, S)` bimodule and `Y` an `R`-module and `Z` an `S`-module
so to use the `Tower` file, we need `S` to be an `R`-algebra which is a luxury we do not have.
But note that in `Tower` file, `curry` and `uncurry` are both tri-linear maps. So `Tower` file
allows interplay of 3 rings which is not allowed in this file.
2. We require `R` to be commutative but we never used anything commutative. This is because of tensor product requires commutativity, but thanks to @alreadydone, this assumption could be removed soon.
I think this PR should wait for Junyan's attempt on removing commutativity, so it is marked as draft and wip for now
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
awaiting-author
WIP
label:t-algebra$ |
214/0 |
Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/TensorHomAdjunction.lean |
2 |
88 |
['alreadydone', 'bustercopley', 'eric-wieser', 'github-actions', 'jjaassoonn', 'kbuzzard', 'kim-em', 'leanprover-community-bot-assistant'] |
eric-wieser assignee:eric-wieser |
118-72927 3 months ago |
118-72928 3 months ago |
0-0 0 seconds |
19284 |
adomani author:adomani |
test: commit a change only to the "master" CI build action |
This PR should fail CI, since the main CI build file is incompatible with the autogenerated ones.
---
[](https://gitpod.io/from-referrer/)
|
CI
merge-conflict
awaiting-author
|
3/3 |
.github/build.in.yml,.github/workflows/actionlint.yml |
2 |
12 |
['adomani', 'bryangingechen', 'github-actions', 'jcommelin', 'leanprover-community-bot-assistant'] |
bryangingechen assignee:bryangingechen |
117-17931 3 months ago |
117-17932 3 months ago |
0-0 0 seconds |
15651 |
TpmKranz author:TpmKranz |
feat(Computability/NFA): operations for Thompson's construction |
Lays the groundwork for a proof of equivalence of RE and NFA, w.r.t. described language. Actual connection to REs comes later, after the groundwork for the opposite direction has been laid.
Third chunk of #12648
---
[](https://gitpod.io/from-referrer/)
|
awaiting-zulip
t-computability
new-contributor
merge-conflict
awaiting-author
|
307/5 |
Mathlib/Computability/NFA.lean |
1 |
15 |
['TpmKranz', 'YaelDillies', 'dupuisf', 'github-actions', 'leanprover-community-bot-assistant', 'meithecatte'] |
nobody |
116-66643 3 months ago |
116-66644 3 months ago |
45-84611 45 days |
22361 |
rudynicolop author:rudynicolop |
feat(Computability/NFA): nfa closure properties |
Add the closure properties union, intersection and reversal for NFA.
---
[](https://gitpod.io/from-referrer/)
|
awaiting-zulip
t-computability
new-contributor
merge-conflict
awaiting-author
|
218/2 |
Mathlib/Computability/Language.lean,Mathlib/Computability/NFA.lean |
2 |
90 |
['EtienneC30', 'b-mehta', 'github-actions', 'leanprover-community-bot-assistant', 'meithecatte', 'rudynicolop'] |
EtienneC30 assignee:EtienneC30 |
116-65717 3 months ago |
116-65719 3 months ago |
39-67601 39 days |
15254 |
yuma-mizuno author:yuma-mizuno |
feat(CategoryTheory/Monoidal): replace `Mon_` lemmas with `Mon_Class` lemmas |
We redefine algebras internal to monoidal categories, which were defined by full-bundled structures, in terms of semi-bundled type classes. The original full-bundled structure `X` is renamed to `X_Cat`.
---
[](https://gitpod.io/from-referrer/)
|
t-category-theory
merge-conflict
WIP
|
3982/96 |
Mathlib.lean,Mathlib/CategoryTheory/Monoidal/Bimod_Class.lean,Mathlib/CategoryTheory/Monoidal/Bimon_.lean,Mathlib/CategoryTheory/Monoidal/Bimon_Class copy.lean,Mathlib/CategoryTheory/Monoidal/Bimon_Class.lean,Mathlib/CategoryTheory/Monoidal/Braided/Opposite.lean,Mathlib/CategoryTheory/Monoidal/CommMon_Class.lean,Mathlib/CategoryTheory/Monoidal/Comon_.lean,Mathlib/CategoryTheory/Monoidal/Comon_Class.lean,Mathlib/CategoryTheory/Monoidal/Internal/ModuleClass.lean,Mathlib/CategoryTheory/Monoidal/Mod_Class.lean,Mathlib/CategoryTheory/Monoidal/Mon_.lean,Mathlib/CategoryTheory/Monoidal/Mon_Class.lean,Mathlib/CategoryTheory/Monoidal/mwe.lean |
14 |
n/a |
['YaelDillies', 'github-actions', 'leanprover-community-bot-assistant', 'yuma-mizuno'] |
nobody |
113-43502 3 months ago |
unknown |
unknown |
22837 |
joneugster author:joneugster |
feat(Data/Set/Basic): add subset_iff and not_mem_subset_iff |
Add `Set.subset_iff` for consistent API with `Finset.subset_iff`.
Add `Set.not_mem_subset_iff` and `Finset.not_mem_subset_iff`.
---
[](https://gitpod.io/from-referrer/)
|
t-set-theory
t-data
merge-conflict
|
9/0 |
Mathlib/Data/Finset/Defs.lean,Mathlib/Data/Set/Basic.lean |
2 |
4 |
['Ruben-VandeVelde', 'github-actions', 'joneugster', 'leanprover-community-bot-assistant'] |
nobody |
110-74739 3 months ago |
110-74741 3 months ago |
30-35190 30 days |
23489 |
plp127 author:plp127 |
chore: fix recursors |
Replace motive with `motive` and other improvements. Will probably split this PR after fixing is done.
4013 recursors left
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict
WIP
|
4255/172 |
Mathlib/Algebra/EuclideanDomain/Basic.lean,Mathlib/Algebra/EuclideanDomain/Defs.lean,Mathlib/Algebra/Free.lean,Mathlib/Algebra/FreeMonoid/Basic.lean,Mathlib/Algebra/Group/Defs.lean,Mathlib/Algebra/Lie/BaseChange.lean,Mathlib/Algebra/Lie/IdealOperations.lean,Mathlib/Algebra/Lie/TraceForm.lean,Mathlib/Algebra/Order/Rearrangement.lean,Mathlib/Algebra/Ring/Subsemiring/Basic.lean,Mathlib/AlgebraicTopology/SimplexCategory/GeneratorsRelations/Basic.lean,Mathlib/Analysis/BoxIntegral/Partition/SubboxInduction.lean,Mathlib/CategoryTheory/Quotient.lean,Mathlib/Data/Fin/Basic.lean,Mathlib/Data/Fin/Tuple/Basic.lean,Mathlib/Data/Fin/Tuple/BubbleSortInduction.lean,Mathlib/Data/Fin/Tuple/NatAntidiagonal.lean,Mathlib/Data/FinEnum/Option.lean,Mathlib/Data/Finset/Max.lean,Mathlib/Data/Fintype/CardEmbedding.lean,Mathlib/Data/Fintype/Option.lean,Mathlib/Data/NNRat/Defs.lean,Mathlib/Data/Nat/BinaryRec.lean,Mathlib/Data/PFun.lean,Mathlib/Data/PFunctor/Multivariate/W.lean,Mathlib/Data/Quot.lean,Mathlib/Data/Sym/Sym2.lean,Mathlib/GroupTheory/Congruence/Defs.lean,Mathlib/GroupTheory/Coprod/Basic.lean,Mathlib/GroupTheory/Coset/Defs.lean,Mathlib/GroupTheory/Coxeter/Basic.lean,Mathlib/LinearAlgebra/Span/Defs.lean,Mathlib/LinearAlgebra/TensorProduct/Tower.lean,Mathlib/NumberTheory/LSeries/HurwitzZetaEven.lean,Mathlib/NumberTheory/LSeries/HurwitzZetaOdd.lean,Mathlib/Order/DirectedInverseSystem.lean,Mathlib/RingTheory/AdicCompletion/Basic.lean,Mathlib/SetTheory/Cardinal/Defs.lean,Mathlib/SetTheory/PGame/Algebra.lean,done.csv,print.lean,working.csv |
42 |
3 |
['github-actions', 'leanprover-community-bot-assistant'] |
nobody |
110-74220 3 months ago |
110-74221 3 months ago |
0-0 0 seconds |
24100 |
eric-wieser author:eric-wieser |
feat: restore some explicit binders from Lean 3 |
Part of #24099
---
[](https://gitpod.io/from-referrer/)
|
tech debt
merge-conflict
awaiting-author
|
39/42 |
Mathlib/Data/FinEnum.lean,Mathlib/FieldTheory/Galois/Profinite.lean,Mathlib/Topology/Bases.lean,Mathlib/Topology/Compactness/CompactlyGeneratedSpace.lean,Mathlib/Topology/MetricSpace/IsometricSMul.lean,Mathlib/Topology/Metrizable/CompletelyMetrizable.lean,Mathlib/Topology/Metrizable/Uniformity.lean,Mathlib/Topology/Order.lean,Mathlib/Topology/Order/LowerUpperTopology.lean,Mathlib/Topology/UniformSpace/UniformEmbedding.lean |
10 |
3 |
['github-actions', 'grunweg', 'leanprover-community-bot-assistant'] |
nobody |
110-74095 3 months ago |
110-74097 3 months ago |
34-33204 34 days |
21476 |
grunweg author:grunweg |
feat(lint-style): enable running on downstream projects |
Enable lint-style to run on downstream projects, by making the following modifications:
- allow passing an explicit list of libraries to lint: if nothing is passed, it lints `Mathlib`, `Archive` and `Counterexamples` (as before); otherwise, it lints precisely the passed modules
- only check init imports, undocumented scripts and the errors from `lint-style.py` when linting Mathlib
- make the style exceptions file configurable and optional: using the `nolints-file` flag, the exceptions file can be configured. If the flag is omitted, we try to find a file at `scripts/nolints-style.txt` --- and otherwise proceed with no style exceptions.
This means mathlib can continue unchanged, and downstream projects can either add an explicit exceptions file, or proceed without any exceptions.
After this PR, one should be able to run lint-style on a downstream project by `lake exe lint-style ProjectName`.
Prompted by [this zulip discussion](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/lint-style.20for.20downstream.20libraries).
---
- [ ] depends on: #24570
- [ ] depends on: #24953
(I did not test the last part.)
[](https://gitpod.io/from-referrer/)
|
t-linter
merge-conflict
|
58/19 |
Mathlib/Tactic/Linter/TextBased.lean,scripts/lint-style.lean |
2 |
19 |
['Vierkantor', 'adomani', 'github-actions', 'grunweg', 'joneugster', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
joneugster assignee:joneugster |
109-80227 3 months ago |
109-80230 3 months ago |
43-17409 43 days |
24163 |
urkud author:urkud |
refactor(TangentCone): redefine for TVS |
---
[](https://gitpod.io/from-referrer/)
|
t-analysis
merge-conflict
|
421/284 |
Mathlib/Analysis/Calculus/FDeriv/Basic.lean,Mathlib/Analysis/Calculus/TangentCone.lean,Mathlib/Topology/Algebra/ConstMulAction.lean |
3 |
4 |
['github-actions', 'leanprover-community-bot-assistant'] |
nobody |
109-25544 3 months ago |
109-25545 3 months ago |
0-0 0 seconds |
23349 |
BGuillemet author:BGuillemet |
feat: add LocallyLipschitzOn.lipschitzOnWith_of_isCompact and two small lemmas about Lipschitz functions |
Main feat (in Mathlib/Topology/EMetricSpace/Basic.lean): if a function `f` from an extended pseudometric space to a pseudometric space is locally Lipschitz on a compact subset `s`, then `f` is Lipschitz on `s`. The theorem is true only when the codomain of `f` is a pseudometric space, so it needs imports from Mathlib/Topology/MetricSpace.
Other small feat (in Mathlib/Analysis/Calculus/ContDiff/RCLike.lean): a function that is continuously differentiable on an open subset is locally Lipschitz on this subset.
---
- [ ] depends on: #22890
[](https://gitpod.io/from-referrer/)
|
large-import
new-contributor
t-topology
merge-conflict
|
59/4 |
Mathlib/Analysis/Calculus/ContDiff/RCLike.lean,Mathlib/Topology/EMetricSpace/Lipschitz.lean |
2 |
4 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
PatrickMassot assignee:PatrickMassot |
108-61957 3 months ago |
108-61959 3 months ago |
35-30364 35 days |
23767 |
grunweg author:grunweg |
refactor: make library notes a definition |
Make library notes a definition of `Unit` type, whose doc-string is the note's content. As a consequence,
- doc-gen will display all library notes without any custom logic,
- library notes are shown upon hover (via the use of the doc-string),
- go do definition for library notes is easy
Automate this using a macro, which also enforces that all library notes are inside the Mathlib.LibraryNote namespace.
*Temporarily*, we use the `library_note2` name; if/when the batteries version is changed, we can reclaim the original name.
This PR does not address how to *refer* to library notes nicely (in a way that is shown in the documentation, checked for typos, with sufficient imports ensured etc.). That is left to a future PR.
This is proposal 2a from this [zulip discussion]([#mathlib4 > library notes @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/library.20notes/near/510614740))
------------
Open questions/TODOs:
- should this go in batteries instead? can the old definition just be overwritten?
- otherwise, what's the best place for the `LibraryNote` definition? A single file just for this feels overkill; I put it in Mathlib.Tactic.Basic for now. I could use Mathlib.Init, of course (but that might be excessive)
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-meta
merge-conflict
|
48/48 |
Archive/Imo/Imo2019Q2.lean,Mathlib/Algebra/BigOperators/Group/Finset/Defs.lean,Mathlib/Algebra/Category/Ring/Limits.lean,Mathlib/Algebra/Group/Action/Defs.lean,Mathlib/Algebra/Group/Conj.lean,Mathlib/Algebra/Group/Defs.lean,Mathlib/Algebra/Group/Hom/Defs.lean,Mathlib/Algebra/Group/Pointwise/Set/Basic.lean,Mathlib/Algebra/Group/Pointwise/Set/Scalar.lean,Mathlib/Algebra/Group/Submonoid/Operations.lean,Mathlib/Algebra/HierarchyDesign.lean,Mathlib/Algebra/Order/Hom/Basic.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Note.lean,Mathlib/Analysis/RCLike/Lemmas.lean,Mathlib/CategoryTheory/Category/Basic.lean,Mathlib/Data/NNRat/Defs.lean,Mathlib/Data/Nat/Cast/Defs.lean,Mathlib/Data/Nat/Init.lean,Mathlib/Geometry/Manifold/Algebra/Monoid.lean,Mathlib/Geometry/Manifold/ChartedSpace.lean,Mathlib/Logic/Basic.lean,Mathlib/Tactic/Basic.lean,Mathlib/Tactic/NormNum/Basic.lean,Mathlib/Tactic/Simps/Basic.lean,Mathlib/Topology/Algebra/Nonarchimedean/Bases.lean,Mathlib/Topology/Continuous.lean |
26 |
9 |
['adomani', 'github-actions', 'grunweg', 'leanprover-community-bot-assistant'] |
nobody |
106-75052 3 months ago |
106-75054 3 months ago |
51-69759 51 days |
12438 |
jjaassoonn author:jjaassoonn |
feat: some APIs for flat modules |
Need horseshoe lemma
---
[](https://gitpod.io/from-referrer/)
|
t-category-theory
merge-conflict
WIP
|
1674/3 |
Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Monoidal/Basic.lean,Mathlib/Algebra/Category/ModuleCat/Monoidal/Symmetric.lean,Mathlib/Algebra/Exact.lean,Mathlib/CategoryTheory/Abelian/Basic.lean,Mathlib/CategoryTheory/Abelian/DiagramLemmas/Horseshoe.lean,Mathlib/CategoryTheory/Abelian/LeftDerived.lean,Mathlib/RingTheory/Flat/Basic.lean |
8 |
21 |
['erdOne', 'github-actions', 'jjaassoonn', 'joelriou'] |
nobody |
103-74583 3 months ago |
490-5600 1 year ago |
0-0 0 seconds |
24965 |
erdOne author:erdOne |
refactor: Make `IsLocalHom` take unbundled map |
---
[](https://gitpod.io/from-referrer/)
|
maintainer-merge
t-algebra
merge-conflict
awaiting-author
label:t-algebra$ |
16/7 |
Mathlib/Algebra/Group/Units/Hom.lean,Mathlib/AlgebraicGeometry/Scheme.lean,Mathlib/Geometry/RingedSpace/LocallyRingedSpace.lean,Mathlib/Geometry/RingedSpace/LocallyRingedSpace/HasColimits.lean,Mathlib/Geometry/RingedSpace/OpenImmersion.lean |
5 |
6 |
['alreadydone', 'erdOne', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant'] |
nobody |
102-28938 3 months ago |
102-28939 3 months ago |
10-26015 10 days |
8740 |
digama0 author:digama0 |
fix: improve `recall` impl / error reporting |
Simplifies the implementation of `recall`, fixing a bug [reported on Zulip](https://leanprover.zulipchat.com/#narrow/stream/113488-general/topic/.60recall.60.20strangeness/near/405076713) and also eliminating a use of `open private`.
---
[](https://gitpod.io/from-referrer/)
|
awaiting-CI
t-meta
merge-conflict
awaiting-author
|
27/39 |
Mathlib/Tactic/Recall.lean |
1 |
2 |
['github-actions', 'leanprover-community-bot-assistant'] |
nobody |
102-5444 3 months ago |
102-5446 3 months ago |
0-0 0 seconds |
21182 |
joneugster author:joneugster |
fix(Util/CountHeartbeats): move elaboration in #count_heartbeats inside a namespace |
Currently the `#count_heartbeat` linter reported the heartbeats until it concluded `error: [declaration] has already been declared` instead of re-elaborating the declaration.
---
[Zulip report](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/count_heartbeats.20for.20all.20declarations.20in.20a.20file.3F/near/496303652)
[](https://gitpod.io/from-referrer/)
|
t-meta
merge-conflict
|
72/5 |
Mathlib/Util/CountHeartbeats.lean,MathlibTest/CountHeartbeats.lean |
2 |
17 |
['adomani', 'github-actions', 'joneugster', 'leanprover-community-bot-assistant', 'mathlib-bors'] |
adomani assignee:adomani |
102-4305 3 months ago |
102-4306 3 months ago |
64-19141 64 days |
17715 |
adomani author:adomani |
feat: the unusedVariableCommand linter |
This is still work-in-progress, but also help-wanted!
The linter reliably flags unused variables: so far, only `example`s fool it (and that is simply because I did not implement a fix, as there are very few `variable`s that are only used in `example`s in mathlib).
The work-in-progress part refers to the fact that the linter uses an `IO.Ref` to keep track of variables and this does not work well with editing the file. The linter works on a fresh parse of a file, but becomes out-of-sync with every edit.
The help-wanted is to ask for help to make mathlib compliant with the linter, by checking out this branch and PR-ing a few variable removals!
[Zulip discussion](https://leanprover.zulipchat.com/#narrow/stream/113488-general/topic/Unused.20variables)
---
Known issues:
* automatic namespacing and `nonrec` may cause difficulty when the newly introduced declaration is preferred in the term, rather than the original one (see examples here
```bash
code -r -g ././././Mathlib/Analysis/SpecialFunctions/Arsinh.lean:183
code -r -g ././././Mathlib/Probability/Independence/Basic.lean:368
```
where, for instance, `ContinuousOn.arsinh` is used internally instead of `Real.arsinh`).
* `mutual` declarations confuse the linter
```bash
code -r -g ././././Mathlib/SetTheory/Lists.lean:313
```
* `code -r -g Mathlib/CategoryTheory/EffectiveEpi/Comp.lean:133:29`
* universe annotations confuse the linter:
```bash
code -r -g ././././Mathlib/Topology/Category/CompactlyGenerated.lean:53
code -r -g ././././Mathlib/AlgebraicTopology/CechNerve.lean:46
```
* `inductive`s confusing the linter
```bash
code -r -g ././././Mathlib/Deprecated/Subgroup.lean:389
code -r -g ././././Mathlib/FieldTheory/PerfectClosure.lean:55
```
* `def`s confusing the linter
```bash
code -r -g ././././Mathlib/Data/MLList/BestFirst.lean:104
```
* special typeclass assumptions
```code
code -r -g ././././Mathlib/RingTheory/WittVector/Truncated.lean:273
code -r -g ././././Mathlib/Topology/Category/Profinite/Product.lean:79
```
* not sure what is going on here:
```bash
code -r -g ././././Mathlib/RingTheory/WittVector/IsPoly.lean:95
code -r -g ././././Mathlib/Probability/Independence/Basic.lean:368
code -r -g ././././Mathlib/Analysis/Calculus/FDeriv/Star.lean:30
```
[](https://gitpod.io/from-referrer/)
|
large-import
t-linter
merge-conflict
|
695/22 |
Mathlib.lean,Mathlib/Algebra/Group/Idempotent.lean,Mathlib/Algebra/GroupWithZero/Idempotent.lean,Mathlib/Data/Finite/Defs.lean,Mathlib/Data/Int/Cast/Field.lean,Mathlib/Geometry/Manifold/IntegralCurve/ExistUnique.lean,Mathlib/Init.lean,Mathlib/MeasureTheory/Function/LpSpace/DomAct/Continuous.lean,Mathlib/NumberTheory/LSeries/PrimesInAP.lean,Mathlib/Order/BoundedOrder/Basic.lean,Mathlib/Order/BoundedOrder/Lattice.lean,Mathlib/Order/BoundedOrder/Monotone.lean,Mathlib/Order/Monotone/Monovary.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter/UnusedVariableCommand.lean,MathlibTest/UnusedVariableCommand.lean,lakefile.lean |
17 |
n/a |
['github-actions', 'grunweg', 'leanprover-community-bot-assistant'] |
nobody |
101-69341 3 months ago |
unknown |
unknown |
24105 |
urkud author:urkud |
feat(Topology/UniformSpace/Path): new file |
---
- [x] depends on: #24066
[](https://gitpod.io/from-referrer/)
|
t-topology
merge-conflict
awaiting-author
|
117/5 |
Mathlib.lean,Mathlib/Topology/ContinuousMap/Defs.lean,Mathlib/Topology/Order/ProjIcc.lean,Mathlib/Topology/Path.lean,Mathlib/Topology/UniformSpace/CompactConvergence.lean,Mathlib/Topology/UniformSpace/Path.lean |
6 |
10 |
['ADedecker', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'sgouezel', 'urkud'] |
nobody |
101-63724 3 months ago |
101-63725 3 months ago |
12-77412 12 days |
23371 |
grunweg author:grunweg |
chore: mark `Disjoint.{eq_bot, inter_eq}` simp |
And add the analogous lemma to `Finset`.
Spun out from #22964, hence transitively part of my bordism theory project.
Some lemmas there are more conveniently stated with `Disjoint`, which requires tagging at least `inter_eq` with simp.
---
[](https://gitpod.io/from-referrer/)
|
t-order
merge-conflict
awaiting-author
|
12/11 |
Mathlib/Data/Finset/Lattice/Basic.lean,Mathlib/Data/Finset/Lattice/Lemmas.lean,Mathlib/Data/Set/Basic.lean,Mathlib/Data/Set/Disjoint.lean,Mathlib/Order/Disjoint.lean,Mathlib/Topology/Compactification/OnePoint.lean,Mathlib/Topology/Order/OrderClosed.lean |
7 |
31 |
['YaelDillies', 'eric-wieser', 'github-actions', 'grunweg', 'j-loreaux', 'leanprover-bot', 'leanprover-community-bot-assistant', 'leanprover-community-mathlib4-bot'] |
nobody |
100-75066 3 months ago |
100-75069 3 months ago |
32-65400 32 days |
16020 |
adomani author:adomani |
feat: compare PR `olean`s size with `master` |
Adds two CI steps:
* `print the sizes of the oleans` that prints the sizes of all the folders containing `Mathlib` `.olean`s;
* `compare oleans` that compares the sizes of the previous step with the corresponding sizes on `master`.
In the test runs, the two steps have taken at most 3 seconds combined (the first is virtually instantaneous, the second one depends on `curl` to find a job id and on `gh` to retrieve the logs of a previous CI run -- everything else appears to be negligible).
This hopefully helps finding out if some PR is bloating up the `.olean`s.
See [this Zulip discussion](https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/Error.3A.20No.20space.20left.20on.20device/near/463792355) for a PR of mine that prompted this check.
---
[](https://gitpod.io/from-referrer/)
|
CI
merge-conflict
|
120/0 |
.github/build.in.yml,.github/workflows/bors.yml,.github/workflows/build.yml,.github/workflows/build_fork.yml,scripts/olean_comparison.sh |
5 |
50 |
['Vtec234', 'YaelDillies', 'adomani', 'bryangingechen', 'github-actions', 'grunweg', 'kim-em', 'leanprover-community-bot-assistant', 'mattrobball'] |
nobody |
99-25564 3 months ago |
99-25566 3 months ago |
285-26861 285 days |
16062 |
adomani author:adomani |
Test/ci olean size |
Tests for oleans
---
[](https://gitpod.io/from-referrer/)
|
CI
merge-conflict
awaiting-author
WIP
|
114/0 |
.github/build.in.yml,.github/workflows/bors.yml,.github/workflows/build.yml,.github/workflows/build_fork.yml,scripts/olean_comparison.sh |
5 |
4 |
['Parcly-Taxel', 'adomani', 'github-actions', 'leanprover-community-bot-assistant'] |
nobody |
99-25564 3 months ago |
99-25565 3 months ago |
0-16 16 seconds |
25507 |
eric-wieser author:eric-wieser |
chore(RingTheory/Valuation): golf using `Con` |
This has no particular motivation besides seeing if `Con` is a performant substitute.
---
[](https://gitpod.io/from-referrer/)
|
bench-after-CI
t-algebra
merge-conflict
label:t-algebra$ |
20/35 |
Mathlib/RingTheory/Valuation/ValuationRing.lean |
1 |
2 |
['github-actions', 'leanprover-community-bot-assistant'] |
nobody |
99-17043 3 months ago |
99-17044 3 months ago |
0-0 0 seconds |
12799 |
jstoobysmith author:jstoobysmith |
feat(LinearAlgebra/UnitaryGroup): Add properties of Special Unitary Group |
Add properties of the special unitary group, mirroring the properties of found in Algebra/Star/Unitary.lean. In particular, I add an instance of `specialUnitaryGroup` as a `Group`, `Star`, `InvolutiveStar`, and `StarMul`.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-algebra
merge-conflict
please-adopt
awaiting-author
label:t-algebra$ |
78/0 |
Mathlib/LinearAlgebra/UnitaryGroup.lean |
1 |
8 |
['chrisflav', 'jcommelin', 'leanprover-community-bot-assistant'] |
nobody |
98-33910 3 months ago |
98-33912 3 months ago |
9-22007 9 days |
23709 |
plp127 author:plp127 |
feat: `Nat.findFrom` |
This PR adds `Nat.findFrom`, which is like `Nat.find`, but starting from an arbitrary `k` instead of `0`.
---
[](https://gitpod.io/from-referrer/)
|
t-data
merge-conflict
|
190/47 |
Mathlib/Data/Nat/Find.lean |
1 |
2 |
['github-actions', 'leanprover-community-bot-assistant'] |
nobody |
97-85599 3 months ago |
97-85601 3 months ago |
62-25661 62 days |
25340 |
dupuisf author:dupuisf |
chore(Analysis/Convex): move files pertaining to convex/concave functions to their own folder |
This PR creates a new folder under `Analysis/Convex` called `Analysis/Convex/Function`, which includes files that are mostly or entirely about convex/concave functions (as opposed to convex sets).
---
[](https://gitpod.io/from-referrer/)
|
t-convex-geometry
merge-conflict
|
4264/4155 |
Mathlib.lean,Mathlib/Analysis/Convex/Continuous.lean,Mathlib/Analysis/Convex/Deriv.lean,Mathlib/Analysis/Convex/Exposed.lean,Mathlib/Analysis/Convex/Extrema.lean,Mathlib/Analysis/Convex/Function.lean,Mathlib/Analysis/Convex/Function/Basic.lean,Mathlib/Analysis/Convex/Function/Continuous.lean,Mathlib/Analysis/Convex/Function/Deriv.lean,Mathlib/Analysis/Convex/Function/Extrema.lean,Mathlib/Analysis/Convex/Function/Integral.lean,Mathlib/Analysis/Convex/Function/Jensen.lean,Mathlib/Analysis/Convex/Function/Mul.lean,Mathlib/Analysis/Convex/Function/Piecewise.lean,Mathlib/Analysis/Convex/Function/Quasiconvex.lean,Mathlib/Analysis/Convex/Function/Slope.lean,Mathlib/Analysis/Convex/Function/Strong.lean,Mathlib/Analysis/Convex/Integral.lean,Mathlib/Analysis/Convex/Jensen.lean,Mathlib/Analysis/Convex/Mul.lean,Mathlib/Analysis/Convex/Piecewise.lean,Mathlib/Analysis/Convex/Quasiconvex.lean,Mathlib/Analysis/Convex/Slope.lean,Mathlib/Analysis/Convex/SpecificFunctions/Basic.lean,Mathlib/Analysis/Convex/SpecificFunctions/Deriv.lean,Mathlib/Analysis/Convex/Strong.lean,Mathlib/Analysis/MeanInequalities.lean,Mathlib/Analysis/MeanInequalitiesPow.lean,Mathlib/Analysis/Normed/Module/Convex.lean,Mathlib/Analysis/Seminorm.lean,Mathlib/Analysis/SpecialFunctions/Log/NegMulLog.lean,Mathlib/Analysis/SpecialFunctions/Pochhammer.lean,Mathlib/MeasureTheory/Measure/Decomposition/IntegralRNDeriv.lean,Mathlib/NumberTheory/Harmonic/GammaDeriv.lean |
34 |
2 |
['github-actions', 'leanprover-community-bot-assistant'] |
nobody |
97-84784 3 months ago |
97-84786 3 months ago |
6-40169 6 days |
13994 |
grunweg author:grunweg |
chore(Topology): replace continuity -> fun_prop |
Addresses a few porting notes; I expect also a substantial speed-up of some proofs.
Change a few default values of proof fields from `continuity` to `fun_prop`; this required a few fix-ups downstream. (I checked a few instances; the failure seems related to `Continuous.subtype_mk` not always firing.)
This is almost (but not fully) exhaustive.
----------
One proof gets partially un-automated (cont. -> partial fun_prop); if desired, I can revert this change.
- [x] depends on: #11092
[](https://gitpod.io/from-referrer/)
|
t-topology
merge-conflict
|
105/20 |
Mathlib/Analysis/Distribution/FourierSchwartz.lean,Mathlib/Analysis/Matrix.lean,Mathlib/Dynamics/Flow.lean,Mathlib/Geometry/RingedSpace/OpenImmersion.lean,Mathlib/Topology/Algebra/Field.lean,Mathlib/Topology/Algebra/Monoid.lean,Mathlib/Topology/Category/TopCat/Limits/Basic.lean,Mathlib/Topology/Category/TopCat/Limits/Pullbacks.lean,Mathlib/Topology/ContinuousMap/Basic.lean,Mathlib/Topology/ContinuousMap/Bounded/Basic.lean,Mathlib/Topology/ContinuousMap/Compact.lean,Mathlib/Topology/ContinuousMap/StoneWeierstrass.lean,Mathlib/Topology/ExtremallyDisconnected.lean,Mathlib/Topology/Homotopy/HomotopyGroup.lean,Mathlib/Topology/Homotopy/Path.lean,Mathlib/Topology/Instances/RealVectorSpace.lean,Mathlib/Topology/MetricSpace/Perfect.lean,Mathlib/Topology/UnitInterval.lean |
18 |
12 |
['MichaelStollBayreuth', 'github-actions', 'grunweg', 'j-loreaux', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'urkud'] |
nobody |
97-17057 3 months ago |
372-36688 1 year ago |
28-21477 28 days |
21734 |
adomani author:adomani |
fix(PR summary): checkout GITHUB_SHA |
This should make the version of the script that is used on PRs more stable.
Suggested by Eric Wieser on [Zulip](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/messageFile.2Emd/near/498941855).
---
[](https://gitpod.io/from-referrer/)
|
CI
merge-conflict
awaiting-author
WIP
|
2/1 |
.github/workflows/PR_summary.yml |
1 |
2 |
['github-actions', 'leanprover-community-bot-assistant'] |
nobody |
97-15051 3 months ago |
97-15053 3 months ago |
0-6023 1 hour |
25012 |
urkud author:urkud |
refactor(*): migrate from `Matrix.toLin'` to `Matrix.mulVecLin` |
or `Matrix.mulVec` whenever we don't need the `LinearEquiv.symm` part.
See [Zulip discussion](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Matrix.2EtoLin'.20vs.20Matrix.2EmulVecLin/with/515188548).
It makes sense to have only one normal form, and `Matrix.toLin'` has an extra `DecidableEq` assumption.
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict |
154/122 |
Mathlib/Algebra/Lie/Matrix.lean,Mathlib/Algebra/Module/Equiv/Basic.lean,Mathlib/Analysis/CStarAlgebra/Matrix.lean,Mathlib/Analysis/Matrix.lean,Mathlib/Combinatorics/SimpleGraph/LapMatrix.lean,Mathlib/Data/Matrix/Rank.lean,Mathlib/LinearAlgebra/Basis/Defs.lean,Mathlib/LinearAlgebra/Determinant.lean,Mathlib/LinearAlgebra/Finsupp/VectorSpace.lean,Mathlib/LinearAlgebra/FreeModule/Finite/Matrix.lean,Mathlib/LinearAlgebra/Matrix/BilinearForm.lean,Mathlib/LinearAlgebra/Matrix/Charpoly/Minpoly.lean,Mathlib/LinearAlgebra/Matrix/Diagonal.lean,Mathlib/LinearAlgebra/Matrix/Gershgorin.lean,Mathlib/LinearAlgebra/Matrix/SesquilinearForm.lean,Mathlib/LinearAlgebra/Matrix/SpecialLinearGroup.lean,Mathlib/LinearAlgebra/Matrix/ToLin.lean,Mathlib/LinearAlgebra/Matrix/ToLinearEquiv.lean,Mathlib/LinearAlgebra/UnitaryGroup.lean,Mathlib/MeasureTheory/Measure/Lebesgue/Basic.lean,Mathlib/RingTheory/Smooth/StandardSmooth.lean |
21 |
3 |
['github-actions', 'leanprover-community-bot-assistant'] |
nobody |
96-79618 3 months ago |
96-79620 3 months ago |
15-74981 15 days |
24789 |
Ruben-VandeVelde author:Ruben-VandeVelde |
chore: move Algebra.Group.Hom.End to Algebra.Ring |
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebra
merge-conflict
awaiting-author
label:t-algebra$ |
55/50 |
Mathlib.lean,Mathlib/Algebra/Group/Hom/End.lean,Mathlib/Algebra/Group/Hom/Instances.lean,Mathlib/Algebra/Module/End.lean,Mathlib/Algebra/Ring/Hom/End.lean |
5 |
6 |
['Ruben-VandeVelde', 'YaelDillies', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant'] |
nobody |
95-58483 3 months ago |
95-58485 3 months ago |
0-1530 25 minutes |
13483 |
adomani author:adomani |
feat: automatically replace deprecations |
This PR introduces `lake exe update_deprecations` that uses the cache to automatically replace deprecated declarations with the corresponding un-deprecated one.
The script handles namespacing, replacing a possibly non-fully-qualified, deprecated name with the fully-qualified non-deprecated name.
It is also possible to use
```bash
lake exe update_deprecations --mods One.Two.Three,Dd.Ee.Ff
```
to limit the scope of the replacements to the modules `One.Two.Three` and `Dd.Ee.Ff`.
This is intended to be a first step in automating updates: combining this with a linter that emits appropriate warnings, the functionality of `lake exe update_deprecations` can be extended to perform more complicated updates.
---
[](https://gitpod.io/from-referrer/)
|
t-meta
merge-conflict
delegated
awaiting-author
|
306/0 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/UpdateDeprecations.lean,MathlibTest/UpdateDeprecations.lean,lakefile.lean,scripts/README.md,scripts/update_deprecations.lean |
7 |
16 |
['YaelDillies', 'adomani', 'github-actions', 'j-loreaux', 'jcommelin', 'leanprover-community-bot-assistant', 'mathlib-bors', 'sgouezel'] |
joneugster assignee:joneugster |
94-33786 3 months ago |
94-33787 3 months ago |
34-82472 34 days |
8949 |
sebzim4500 author:sebzim4500 |
Add `by_approx` tactic for proving real inequalities using rational approximation |
feat: Add `by_approx` tactic for proving real inequalities by finding rational approximations
---
```lean
example : |sqrt 2 - 1.414| < 0.001 := by by_approx
```
This is a work in progress, the code is messy and the tactic is often very slow. It also depends on some other PRs that haven't been merged yet.
It currently supports basic operations (`+`, `-`, `*`, `/`, `abs`) and has approximation extensions for `sqrt` and `exp`.
- [ ] depends on: #8167
- [x] depends on: #8832
[](https://gitpod.io/from-referrer/)
|
t-meta
merge-conflict
modifies-tactic-syntax
|
1670/3 |
Mathlib.lean,Mathlib/Data/Int/ModEq.lean,Mathlib/Tactic.lean,Mathlib/Tactic/ByApprox.lean,Mathlib/Tactic/ByApprox/Basic.lean,Mathlib/Tactic/ByApprox/Core.lean,Mathlib/Tactic/ByApprox/Exp.lean,Mathlib/Tactic/ByApprox/Lemmas.lean,Mathlib/Tactic/ByApprox/Test.lean,Mathlib/Tactic/ByApprox/Util.lean,Mathlib/Tactic/GCongr/Core.lean,Mathlib/Tactic/GRW.lean,Mathlib/Tactic/GRW/Core.lean,Mathlib/Tactic/GRW/Lemmas.lean,Mathlib/Tactic/NormNum/NatFactorial.lean,test/ByApprox.lean,test/GRW.lean,test/norm_num_ext.lean |
18 |
1 |
['mathlib4-dependent-issues-bot'] |
nobody |
93-39098 3 months ago |
93-39100 3 months ago |
0-0 0 seconds |
20334 |
miguelmarco author:miguelmarco |
feat: allow polyrith to use a local Singular/Sage install |
Try to call a local install of Singular (either standalone or inside Sage) to find the witness for polyrith before trying to call the online sage cell server.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-meta
merge-conflict
awaiting-author
|
171/48 |
Mathlib/Tactic/Polyrith.lean,scripts/polyrith_sage.py |
2 |
16 |
['eric-wieser', 'github-actions', 'hanwenzhu', 'kim-em', 'miguelmarco', 'mkoeppe'] |
nobody |
91-26463 2 months ago |
211-4425 6 months ago |
27-65384 27 days |
23953 |
b-reinke author:b-reinke |
feat(Data/Matroid/Tutte): define the Tutte polynomial of a matroid |
This PR defines the Tutte polynomial of a matroid and shows basic properties.
- [x] depends on: #23926
- [ ] depends on #24336
- [ ] depends on: #23951
---
[](https://gitpod.io/from-referrer/)
|
t-data
merge-conflict
WIP
|
111/0 |
Mathlib/Algebra/BigOperators/Finprod.lean,Mathlib/Data/Matroid/Tutte/Basic.lean,Mathlib/Data/Set/Image.lean |
3 |
7 |
['apnelson1', 'b-reinke', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
88-67943 2 months ago |
88-67945 2 months ago |
0-0 0 seconds |
18441 |
ADedecker author:ADedecker |
refactor(AdicTopology): use new API for algebraic filter bases, and factor some code |
---
- [x] depends on: #18437
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-topology
merge-conflict
label:t-algebra$ |
847/159 |
Mathlib.lean,Mathlib/Topology/Algebra/FilterBasis.lean,Mathlib/Topology/Algebra/FilterBasisNew.lean,Mathlib/Topology/Algebra/Nonarchimedean/AdicTopology.lean,Mathlib/Topology/Algebra/Nonarchimedean/Bases.lean,Mathlib/Topology/Algebra/Nonarchimedean/BasesNew.lean |
6 |
3 |
['ADedecker', 'github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
85-76525 2 months ago |
85-76527 2 months ago |
0-679 11 minutes |
18439 |
ADedecker author:ADedecker |
refactor: use new algebraic filter bases API in `FiniteAdeleRing` |
---
- [x] depends on: #18437
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-topology
merge-conflict
label:t-algebra$ |
699/21 |
Mathlib.lean,Mathlib/RingTheory/DedekindDomain/FiniteAdeleRing.lean,Mathlib/Topology/Algebra/FilterBasis.lean,Mathlib/Topology/Algebra/FilterBasisNew.lean,Mathlib/Topology/Algebra/Nonarchimedean/Bases.lean,Mathlib/Topology/Algebra/Nonarchimedean/BasesNew.lean |
6 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
85-76523 2 months ago |
85-76525 2 months ago |
0-619 10 minutes |
18438 |
ADedecker author:ADedecker |
refactor: adapt `KrullTopology` to the new algebraic filter bases API |
---
- [x] depends on: #18437
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-topology
merge-conflict
label:t-algebra$ |
771/168 |
Mathlib.lean,Mathlib/FieldTheory/KrullTopology.lean,Mathlib/Topology/Algebra/FilterBasis.lean,Mathlib/Topology/Algebra/FilterBasisNew.lean,Mathlib/Topology/Algebra/Nonarchimedean/Bases.lean,Mathlib/Topology/Algebra/Nonarchimedean/BasesNew.lean |
6 |
5 |
['ADedecker', 'AntoineChambert-Loir', 'github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
85-76522 2 months ago |
85-76523 2 months ago |
0-638 10 minutes |
23040 |
grunweg author:grunweg |
feat: define immersions and smooth embeddings in infinite dimensions |
Sadly, we cannot prove most nice things about them yet, as we don't have
the inverse function theorem yet.
TODO: prove the few things we can already say
---
- [ ] depends on: #23175 (preliminaries)
- [x] depends on: #23186
- [ ] depends on: another PR, about `MSplitAt` (to be filed) - and perhaps some prerequisites about products of complemented modules etc.
- [ ] depends on: #23219 (preliminaries about local diffeomorphisms)
- [ ] depends on: #8738
- in fact, #9273 is not a strict pre-requisite for this. It suffices to know "extended charts have invertible differentials", which [isInvertible_mfderiv_extChartAt](https://leanprover-community.github.io/mathlib4_docs/Mathlib/Geometry/Manifold/MFDeriv/Atlas.html#isInvertible_mfderiv_extChartAt) mostly proves. (There's nothing wrong with completing that PR, for all interior points.)
[](https://gitpod.io/from-referrer/)
|
t-differential-geometry
merge-conflict
WIP
|
967/0 |
Mathlib.lean,Mathlib/Analysis/NormedSpace/HahnBanach/Splits.lean,Mathlib/Geometry/Manifold/IsImmersionEmbedding.lean,Mathlib/Geometry/Manifold/LocalDiffeomorph.lean,Mathlib/Geometry/Manifold/MSplits.lean |
5 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
85-43511 2 months ago |
85-43513 2 months ago |
0-0 0 seconds |
13964 |
pechersky author:pechersky |
feat(Data/DigitExpansion): begin defining variant of reals without rationals |
Based on a de Bruijn 1976 paper.
This file is just the basic definition of a digit expansion. Will be followed up with further constructions.
---
[](https://gitpod.io/from-referrer/)
|
t-data
merge-conflict
|
518/0 |
Mathlib.lean,Mathlib/Data/DigitExpansion/Defs.lean,docs/references.bib |
3 |
11 |
['eric-wieser', 'github-actions', 'kim-em', 'pechersky'] |
dupuisf assignee:dupuisf |
82-58813 2 months ago |
320-85029 10 months ago |
129-57991 129 days |
26581 |
nomeata author:nomeata |
ignore this: Lean pr testing 9124 |
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict |
1723/1362 |
Archive/Arithcc.lean,Archive/Examples/Eisenstein.lean,Archive/Examples/IfNormalization/WithoutAesop.lean,Archive/Imo/Imo1972Q5.lean,Archive/Imo/Imo1975Q1.lean,Archive/Imo/Imo1987Q1.lean,Archive/Imo/Imo1994Q1.lean,Archive/Imo/Imo1998Q2.lean,Archive/Imo/Imo2006Q5.lean,Archive/Imo/Imo2008Q3.lean,Archive/Imo/Imo2024Q1.lean,Archive/Imo/Imo2024Q3.lean,Archive/Imo/Imo2024Q5.lean,Archive/MiuLanguage/DecisionNec.lean,Archive/MiuLanguage/DecisionSuf.lean,Archive/Sensitivity.lean,Archive/Wiedijk100Theorems/AbelRuffini.lean,Archive/Wiedijk100Theorems/AreaOfACircle.lean,Archive/Wiedijk100Theorems/AscendingDescendingSequences.lean,Archive/Wiedijk100Theorems/BallotProblem.lean,Archive/Wiedijk100Theorems/BuffonsNeedle.lean,Archive/Wiedijk100Theorems/CubingACube.lean,Archive/Wiedijk100Theorems/FriendshipGraphs.lean,Archive/Wiedijk100Theorems/Partition.lean,Archive/Wiedijk100Theorems/PerfectNumbers.lean,Archive/Wiedijk100Theorems/SumOfPrimeReciprocalsDiverges.lean,Archive/ZagierTwoSquares.lean,Cache/Lean.lean,Counterexamples/AharoniKorman.lean,Counterexamples/CanonicallyOrderedCommSemiringTwoMul.lean,Counterexamples/CliffordAlgebraNotInjective.lean,Counterexamples/DiscreteTopologyNonDiscreteUniformity.lean,Counterexamples/MapFloor.lean,Counterexamples/MonicNonRegular.lean,Counterexamples/Phillips.lean,Counterexamples/Pseudoelement.lean,Counterexamples/ZeroDivisorsInAddMonoidAlgebras.lean,Mathlib/Algebra/Algebra/NonUnitalSubalgebra.lean,Mathlib/Algebra/Algebra/Operations.lean,Mathlib/Algebra/Algebra/Subalgebra/Operations.lean,Mathlib/Algebra/Algebra/Subalgebra/Pointwise.lean,Mathlib/Algebra/Algebra/Unitization.lean,Mathlib/Algebra/Algebra/ZMod.lean,Mathlib/Algebra/BigOperators/Fin.lean,Mathlib/Algebra/BigOperators/Finprod.lean,Mathlib/Algebra/BigOperators/Group/List/Basic.lean,Mathlib/Algebra/Category/ContinuousCohomology/Basic.lean,Mathlib/Algebra/Category/ModuleCat/Topology/Basic.lean,Mathlib/Algebra/Category/ModuleCat/Topology/Homology.lean,Mathlib/Algebra/Category/MonCat/FilteredColimits.lean,Mathlib/Algebra/Category/Ring/Epi.lean,Mathlib/Algebra/Category/Ring/FinitePresentation.lean,Mathlib/Algebra/Category/Ring/Topology.lean,Mathlib/Algebra/CharP/Basic.lean,Mathlib/Algebra/CharP/Defs.lean,Mathlib/Algebra/Colimit/Module.lean,Mathlib/Algebra/DirectSum/Algebra.lean,Mathlib/Algebra/DirectSum/Ring.lean,Mathlib/Algebra/DualNumber.lean,Mathlib/Algebra/Equiv/TransferInstance.lean,Mathlib/Algebra/GCDMonoid/Finset.lean,Mathlib/Algebra/Group/Action/Basic.lean,Mathlib/Algebra/Group/Basic.lean,Mathlib/Algebra/Group/End.lean,Mathlib/Algebra/Group/Pointwise/Finset/Basic.lean,Mathlib/Algebra/Group/Pointwise/Finset/Scalar.lean,Mathlib/Algebra/Group/Pointwise/Set/Basic.lean,Mathlib/Algebra/Group/Subgroup/Basic.lean,Mathlib/Algebra/GroupWithZero/Action/Defs.lean,Mathlib/Algebra/GroupWithZero/NonZeroDivisors.lean,Mathlib/Algebra/Lie/CartanExists.lean,Mathlib/Algebra/Lie/LieTheorem.lean,Mathlib/Algebra/Lie/Weights/Chain.lean,Mathlib/Algebra/Lie/Weights/RootSystem.lean,Mathlib/Algebra/Module/Equiv/Defs.lean,Mathlib/Algebra/Module/FinitePresentation.lean,Mathlib/Algebra/Module/LinearMap/Defs.lean,Mathlib/Algebra/Module/Presentation/Basic.lean,Mathlib/Algebra/MonoidAlgebra/Defs.lean,Mathlib/Algebra/MonoidAlgebra/ToDirectSum.lean,Mathlib/Algebra/MvPolynomial/Basic.lean,Mathlib/Algebra/MvPolynomial/Equiv.lean,Mathlib/Algebra/MvPolynomial/Eval.lean,Mathlib/Algebra/MvPolynomial/Variables.lean,Mathlib/Algebra/NoZeroSMulDivisors/Defs.lean,Mathlib/Algebra/Order/Antidiag/Pi.lean,Mathlib/Algebra/Order/CauSeq/Completion.lean,Mathlib/Algebra/Order/Field/Power.lean,Mathlib/Algebra/Order/Ring/Unbundled/Rat.lean,Mathlib/Algebra/Polynomial/Bivariate.lean,Mathlib/Algebra/Polynomial/Degree/CardPowDegree.lean,Mathlib/Algebra/Polynomial/HasseDeriv.lean,Mathlib/Algebra/Quaternion.lean,Mathlib/Algebra/Regular/Pi.lean,Mathlib/Algebra/Ring/Basic.lean,Mathlib/Algebra/Ring/CentroidHom.lean,Mathlib/Algebra/Ring/GrindInstances.lean,Mathlib/Algebra/Ring/Int/Defs.lean,Mathlib/Algebra/RingQuot.lean,Mathlib/Algebra/Star/NonUnitalSubalgebra.lean |
567 |
n/a |
[] |
nobody |
73-74638 2 months ago |
unknown |
unknown |
14752 |
AntoineChambert-Loir author:AntoineChambert-Loir |
fix(Topology/Algebra/Valued): repair definition of Valued |
Following a [discussion on Zulip](https://leanprover.zulipchat.com/#narrow/stream/116395-maths/topic/Question.20about.20.60Valued.2Eis_topological_valuation.60), we modify the definition of the field `is_topological_valuation` of `Valued` insisting that the element $\gamma$ showing up there is in the subgroup generated by the image of the valuation map.
Co-authored-by: @faenuccio
- [ ] depends on: #25496 |
t-algebra
t-topology
merge-conflict
WIP
label:t-algebra$ |
1166/301 |
Mathlib.lean,Mathlib/Algebra/GroupWithZero/Range.lean,Mathlib/NumberTheory/NumberField/FinitePlaces.lean,Mathlib/RingTheory/LaurentSeries.lean,Mathlib/RingTheory/Valuation/Basic.lean,Mathlib/RingTheory/Valuation/RankOne.lean,Mathlib/Topology/Algebra/Valued/LocallyCompact.lean,Mathlib/Topology/Algebra/Valued/NormedValued.lean,Mathlib/Topology/Algebra/Valued/ValuationTopology.lean,Mathlib/Topology/Algebra/Valued/ValuedField.lean,Mathlib/Topology/UniformSpace/AbstractCompletion.lean,docs/references.bib |
12 |
28 |
['AntoineChambert-Loir', 'faenuccio', 'github-actions', 'jcommelin', 'kbuzzard', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'riccardobrasca'] |
riccardobrasca assignee:riccardobrasca |
71-65782 2 months ago |
71-65784 2 months ago |
1-33784 1 day |
15213 |
adomani author:adomani |
dev: add Mathlib.Tactic.Linter.ForallIntro |
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-linter
merge-conflict
WIP
|
608/0 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter.lean,Mathlib/Tactic/Linter/ForallIntro.lean,MathlibTest/ForallIntro.lean |
5 |
5 |
['adomani', 'github-actions', 'grunweg', 'leanprover-community-bot-assistant'] |
nobody |
70-26610 2 months ago |
70-26611 2 months ago |
0-0 0 seconds |
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
merge-conflict
|
243/0 |
Mathlib.lean,Mathlib/Combinatorics/SimpleGraph/Planar.lean,Mathlib/Data/CombinatorialMap.lean |
3 |
28 |
['Parcly-Taxel', 'Rida-Hamadani', 'github-actions', 'lambda-fairy', 'leanprover-community-bot-assistant'] |
kmill assignee:kmill |
70-24388 2 months ago |
70-24389 2 months ago |
72-51453 72 days |
16801 |
awainverse author:awainverse |
feat(ModelTheory/Equivalence): The quotient type of formulas modulo a theory |
Defines `FirstOrder.Language.Theory.Formula`: `T.Formula α` is the quotient of `L.Formula α` by
equivalence modulo a theory `T`.
Puts a boolean algebra instance on `T.Formula α`, with `≤` corresponding to implication.
---
- [x] depends on: #16799
- [x] depends on: #16800
[](https://gitpod.io/from-referrer/)
|
t-logic
merge-conflict
awaiting-author
|
174/60 |
Mathlib/ModelTheory/Complexity.lean,Mathlib/ModelTheory/Equivalence.lean,Mathlib/ModelTheory/Types.lean |
3 |
30 |
['YaelDillies', 'awainverse', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'metinersin'] |
YaelDillies assignee:YaelDillies |
70-24387 2 months ago |
70-24387 2 months ago |
29-26213 29 days |
17458 |
urkud author:urkud |
refactor(Algebra/Group): make `IsUnit` a typeclass |
Also change some lemmas to assume `[IsUnit _]` instead of `[Invertible _]`.
Motivated by potential non-defeq diamonds in #14986, see also [Zulip](https://leanprover.zulipchat.com/#narrow/stream/116395-maths/topic/Invertible.20and.20data)
I no longer plan to merge this PR, but I'm going to cherry-pick some changes to a new PR before closing this one.
---
[](https://gitpod.io/from-referrer/)
|
awaiting-zulip
t-algebra
merge-conflict
label:t-algebra$ |
82/72 |
Mathlib/Algebra/CharP/Invertible.lean,Mathlib/Algebra/Group/Invertible/Basic.lean,Mathlib/Algebra/Group/Units/Defs.lean,Mathlib/Algebra/GroupWithZero/Invertible.lean,Mathlib/Algebra/GroupWithZero/Units/Basic.lean,Mathlib/Algebra/Polynomial/Degree/Units.lean,Mathlib/Algebra/Polynomial/Splits.lean,Mathlib/Analysis/Convex/Segment.lean,Mathlib/Analysis/Normed/Affine/Isometry.lean,Mathlib/Analysis/Normed/Ring/Units.lean,Mathlib/CategoryTheory/Linear/Basic.lean,Mathlib/FieldTheory/Finite/Basic.lean,Mathlib/FieldTheory/Separable.lean,Mathlib/FieldTheory/SeparableDegree.lean,Mathlib/GroupTheory/Submonoid/Inverses.lean,Mathlib/LinearAlgebra/AffineSpace/AffineEquiv.lean,Mathlib/LinearAlgebra/AffineSpace/Combination.lean,Mathlib/LinearAlgebra/CliffordAlgebra/Contraction.lean,Mathlib/LinearAlgebra/CliffordAlgebra/Inversion.lean,Mathlib/LinearAlgebra/CliffordAlgebra/SpinGroup.lean,Mathlib/LinearAlgebra/Eigenspace/Minpoly.lean,Mathlib/NumberTheory/MulChar/Basic.lean,Mathlib/RingTheory/Localization/NumDen.lean,Mathlib/RingTheory/Polynomial/Content.lean,Mathlib/RingTheory/Polynomial/GaussLemma.lean,Mathlib/RingTheory/Valuation/Basic.lean |
26 |
12 |
['MichaelStollBayreuth', 'acmepjz', 'eric-wieser', 'github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'urkud'] |
nobody |
70-24386 2 months ago |
70-24386 2 months ago |
0-66650 18 hours |
17627 |
hrmacbeth author:hrmacbeth |
feat: universal properties of vector bundle constructions |
Characterizations for the smoothness of maps into the total spaces of (1) the direct sum of two vector bundles; (2) the pullback of a vector bundle.
This gap in the library was exposed by #17358.
---
- [x] depends on: #22804
[](https://gitpod.io/from-referrer/)
|
t-differential-geometry
merge-conflict
delegated
|
311/9 |
Mathlib/Data/Bundle.lean,Mathlib/Geometry/Manifold/VectorBundle/Basic.lean,Mathlib/Geometry/Manifold/VectorBundle/Pullback.lean,Mathlib/Topology/FiberBundle/Constructions.lean |
4 |
24 |
['PatrickMassot', 'github-actions', 'grunweg', 'hrmacbeth', 'j-loreaux', 'leanprover-community-bot-assistant', 'mathlib-bors', 'mathlib4-dependent-issues-bot', 'sgouezel'] |
grunweg assignee:grunweg |
70-24385 2 months ago |
70-24385 2 months ago |
91-73632 91 days |
19444 |
joelriou author:joelriou |
feat(CategoryTheory/Sites): Equivalence of categories of sheaves with a dense subsite that is 1-hypercover dense |
The main result is that if `F : C₀ ⥤ C` is a dense subsite (relatively to topologies `J₀` and `J`) and `F.IsOneHypercoverDense J₀ J` (for a certain universe `w`), then if a coefficient category `A` has limits of size `w`, the pushforward functor induces an equivalence `Sheaf J A ≌ Sheaf J₀ A`.
We deduce that if `HasSheafify J₀ A`, then `HasSheafify J A` also holds. This was previously known (see `IsDenseSubsite.sheafEquiv` in `Sites.DenseSubsite`) under a somewhat stronger condition about the existence of limits in `A`.
---
- [x] depends on: #19517
- [x] depends on: #19519
This is very much a draft.
[](https://gitpod.io/from-referrer/)
|
t-category-theory
merge-conflict
WIP
|
937/2 |
Mathlib.lean,Mathlib/CategoryTheory/Sites/Continuous.lean,Mathlib/CategoryTheory/Sites/DenseSubsite/Basic.lean,Mathlib/CategoryTheory/Sites/DenseSubsite/OneHypercoverDense.lean,Mathlib/CategoryTheory/Sites/DenseSubsite/SheafEquiv.lean,Mathlib/CategoryTheory/Sites/OneHypercover.lean |
6 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
70-24262 2 months ago |
70-24262 2 months ago |
0-0 0 seconds |
19796 |
peakpoint author:peakpoint |
feat: L'Hopital's rule from within a convex set |
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-analysis
merge-conflict
|
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 |
15 |
['RemyDegenne', 'github-actions', 'leanprover-community-bot-assistant', 'peakpoint', 'sgouezel'] |
sgouezel assignee:sgouezel |
70-24261 2 months ago |
70-24261 2 months ago |
80-57750 80 days |
22928 |
javra author:javra |
feat(CategoryTheory): infrastructure for inclusion morphisms into products in categories with 0-morphisms |
---
[](https://gitpod.io/from-referrer/)
|
t-category-theory
merge-conflict
|
52/14 |
Mathlib/CategoryTheory/Limits/Shapes/BinaryBiproducts.lean,Mathlib/CategoryTheory/Limits/Shapes/Biproducts.lean,Mathlib/CategoryTheory/Limits/Shapes/ZeroMorphisms.lean |
3 |
2 |
['github-actions', 'leanprover-community-bot-assistant'] |
nobody |
70-23880 2 months ago |
70-23881 2 months ago |
112-51866 112 days |
22952 |
eric-wieser author:eric-wieser |
refactor: reimplement `RingQuot` in terms of `RingCon.Quotient` |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
label:t-algebra$ |
157/184 |
Mathlib/Algebra/RingQuot.lean,Mathlib/GroupTheory/Congruence/Basic.lean,Mathlib/RingTheory/Congruence/Basic.lean,Mathlib/RingTheory/Congruence/Defs.lean |
4 |
2 |
['github-actions', 'leanprover-community-bot-assistant'] |
nobody |
70-23879 2 months ago |
70-23880 2 months ago |
0-0 0 seconds |
23637 |
kirilvino author:kirilvino |
feat(Combinatorics/SimpleGraph): every circuit contains a cycle proof |
circuit to cycle proof
---
This PR uses the bypass definition in a new function for closed walks that removes repeated vertices. Then proves if the closed walk given is a circuit, that the result from this function is a cycle. This is then packaged up similar to the existing ToPath definition, creating a way of transforming a circuit into a cycle.
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-combinatorics
merge-conflict
awaiting-author
|
26/0 |
Mathlib/Combinatorics/SimpleGraph/Path.lean |
1 |
9 |
['b-mehta', 'github-actions', 'kirilvino', 'leanprover-community-bot-assistant'] |
nobody |
70-23872 2 months ago |
70-23873 2 months ago |
13-19789 13 days |
23763 |
grunweg author:grunweg |
feat(Linter.openClassical): also lint for Classical declarations as … |
…a local or scoped instance.
---
- [ ] depends on: #23750
[](https://gitpod.io/from-referrer/)
|
t-linter
merge-conflict
|
138/33 |
Mathlib/RingTheory/Perfection.lean,Mathlib/Tactic/Linter/Style.lean,Mathlib/Topology/MetricSpace/GromovHausdorffRealized.lean,MathlibTest/GeneralizeProofs.lean,MathlibTest/LintStyle.lean |
5 |
6 |
['github-actions', 'grunweg', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
70-23872 2 months ago |
70-23872 2 months ago |
82-7297 82 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
merge-conflict
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 |
30 |
['alreadydone', 'erdOne', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
70-23483 2 months ago |
70-23484 2 months ago |
21-66961 21 days |
24489 |
mattrobball author:mattrobball |
test |
|
merge-conflict |
185/152 |
Mathlib/Algebra/GCDMonoid/Nat.lean,Mathlib/Algebra/Group/Defs.lean,Mathlib/Algebra/GroupWithZero/Defs.lean,Mathlib/Algebra/Polynomial/Coeff.lean,Mathlib/Algebra/Polynomial/Eval/Degree.lean,Mathlib/Algebra/Polynomial/Monic.lean,Mathlib/Algebra/Ring/Defs.lean,Mathlib/AlgebraicGeometry/AffineSpace.lean,Mathlib/Analysis/CStarAlgebra/Classes.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Integral.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Isometric.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Unique.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Unital.lean,Mathlib/Analysis/Complex/Polynomial/Basic.lean,Mathlib/Analysis/InnerProductSpace/Adjoint.lean,Mathlib/Analysis/Normed/Algebra/Spectrum.lean,Mathlib/Analysis/NormedSpace/PiTensorProduct/InjectiveSeminorm.lean,Mathlib/Data/Nat/Bitwise.lean,Mathlib/Data/Nat/Choose/Vandermonde.lean,Mathlib/FieldTheory/Galois/Profinite.lean,Mathlib/FieldTheory/IsAlgClosed/Spectrum.lean,Mathlib/FieldTheory/KummerExtension.lean,Mathlib/FieldTheory/KummerPolynomial.lean,Mathlib/GroupTheory/SpecificGroups/Cyclic.lean,Mathlib/GroupTheory/SpecificGroups/Dihedral.lean,Mathlib/GroupTheory/Subgroup/Center.lean,Mathlib/LinearAlgebra/CliffordAlgebra/Basic.lean,Mathlib/LinearAlgebra/CliffordAlgebra/Grading.lean,Mathlib/LinearAlgebra/ExteriorAlgebra/Grading.lean,Mathlib/LinearAlgebra/Matrix/SpecialLinearGroup.lean,Mathlib/LinearAlgebra/PiTensorProduct.lean,Mathlib/LinearAlgebra/RootSystem/Finite/CanonicalBilinear.lean,Mathlib/NumberTheory/NumberField/CanonicalEmbedding/Basic.lean,Mathlib/RepresentationTheory/FDRep.lean,Mathlib/RingTheory/Spectrum/Prime/ChevalleyComplexity.lean,Mathlib/RingTheory/Valuation/ValuationSubring.lean,Mathlib/RingTheory/WittVector/Frobenius.lean,Mathlib/Tactic/Ring/Basic.lean |
38 |
5 |
['github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'mattrobball'] |
nobody |
70-23478 2 months ago |
70-23479 2 months ago |
0-0 0 seconds |
24558 |
mattrobball author:mattrobball |
test |
|
merge-conflict |
32/30 |
Mathlib/Analysis/Analytic/Basic.lean,Mathlib/Analysis/Calculus/ContDiff/Defs.lean,Mathlib/Data/Matroid/Circuit.lean,Mathlib/Data/Matroid/Closure.lean,Mathlib/Data/Matroid/Loop.lean,Mathlib/Data/Set/Insert.lean,Mathlib/FieldTheory/IntermediateField/Adjoin/Basic.lean,Mathlib/Geometry/Euclidean/Angle/Oriented/Affine.lean,Mathlib/Geometry/Euclidean/Angle/Unoriented/Affine.lean,Mathlib/Geometry/Manifold/ContMDiff/Defs.lean,Mathlib/LinearAlgebra/AffineSpace/FiniteDimensional.lean,Mathlib/Order/Cover.lean |
12 |
5 |
['github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'mattrobball'] |
nobody |
70-23477 2 months ago |
70-23477 2 months ago |
0-0 0 seconds |
24614 |
JovanGerb author:JovanGerb |
chore: rename field `inf` to `min` in `Lattice` |
As suggested by @eric-wieser, this PR renames the `sup` and `inf` fields in `Lattice` to `max` and `min`. This means that we now can extend `Lattice` and `LinearOrder` simultaneously without ending up with duplicate fields. This should be implemented in a future PR for existing classes like `CompleteLinearOrder`.
[Zulip discussion](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/.60sup.60.2F.60inf.60.20or.20.60max.60.2F.60min.60.20for.20set.20interval.20lemmas.3F)
---
[](https://gitpod.io/from-referrer/)
|
t-order
merge-conflict
awaiting-author
|
179/185 |
Mathlib/Algebra/Field/Subfield/Basic.lean,Mathlib/Algebra/Group/Subgroup/Lattice.lean,Mathlib/Algebra/Group/Submonoid/Basic.lean,Mathlib/Algebra/Group/Subsemigroup/Basic.lean,Mathlib/Algebra/Lie/Subalgebra.lean,Mathlib/Algebra/Module/Submodule/Lattice.lean,Mathlib/Algebra/Order/Kleene.lean,Mathlib/Algebra/Order/Ring/Idempotent.lean,Mathlib/Algebra/Ring/Subring/Basic.lean,Mathlib/Algebra/Ring/Subsemiring/Basic.lean,Mathlib/Algebra/Tropical/Lattice.lean,Mathlib/AlgebraicGeometry/IdealSheaf/Basic.lean,Mathlib/Analysis/BoxIntegral/Box/Basic.lean,Mathlib/Analysis/BoxIntegral/Partition/Basic.lean,Mathlib/Analysis/Convex/SimplicialComplex/Basic.lean,Mathlib/Analysis/Normed/Group/Seminorm.lean,Mathlib/Analysis/NormedSpace/ENormedSpace.lean,Mathlib/Analysis/NormedSpace/MStructure.lean,Mathlib/Analysis/Seminorm.lean,Mathlib/CategoryTheory/Groupoid/Subgroupoid.lean,Mathlib/CategoryTheory/Sites/Coverage.lean,Mathlib/CategoryTheory/Sites/Grothendieck.lean,Mathlib/CategoryTheory/Sites/Pretopology.lean,Mathlib/CategoryTheory/Sites/Sieves.lean,Mathlib/CategoryTheory/Subobject/Lattice.lean,Mathlib/CategoryTheory/Subpresheaf/Basic.lean,Mathlib/Combinatorics/Digraph/Basic.lean,Mathlib/Combinatorics/SimpleGraph/Basic.lean,Mathlib/Combinatorics/SimpleGraph/Subgraph.lean,Mathlib/Computability/Reduce.lean,Mathlib/Data/DFinsupp/Order.lean,Mathlib/Data/Finset/Lattice/Basic.lean,Mathlib/Data/Finsupp/Order.lean,Mathlib/Data/Multiset/UnionInter.lean,Mathlib/Data/Nat/PartENat.lean,Mathlib/Data/PEquiv.lean,Mathlib/Data/Real/Basic.lean,Mathlib/Data/Semiquot.lean,Mathlib/Data/Set/Basic.lean,Mathlib/Data/Setoid/Basic.lean,Mathlib/Data/Sum/Lattice.lean,Mathlib/Dynamics/Circle/RotationNumber/TranslationNumber.lean,Mathlib/Geometry/Convex/Cone/Basic.lean,Mathlib/Geometry/Manifold/ChartedSpace.lean,Mathlib/GroupTheory/Congruence/Defs.lean,Mathlib/LinearAlgebra/AffineSpace/AffineSubspace/Defs.lean,Mathlib/LinearAlgebra/LinearPMap.lean,Mathlib/MeasureTheory/Function/AEEqFun.lean,Mathlib/MeasureTheory/Function/SimpleFunc.lean,Mathlib/ModelTheory/Substructures.lean,Mathlib/Order/BooleanSubalgebra.lean,Mathlib/Order/Booleanisation.lean,Mathlib/Order/CompleteLattice/Defs.lean,Mathlib/Order/Concept.lean,Mathlib/Order/ConditionallyCompleteLattice/Defs.lean,Mathlib/Order/Copy.lean,Mathlib/Order/Filter/Basic.lean,Mathlib/Order/Filter/Germ/Basic.lean,Mathlib/Order/FixedPoints.lean,Mathlib/Order/GaloisConnection/Basic.lean,Mathlib/Order/Heyting/Basic.lean,Mathlib/Order/Hom/Order.lean,Mathlib/Order/Ideal.lean,Mathlib/Order/Interval/Basic.lean,Mathlib/Order/Lattice.lean,Mathlib/Order/Partition/Finpartition.lean,Mathlib/Order/PropInstances.lean,Mathlib/Order/Sublattice.lean,Mathlib/Order/WithBot.lean,Mathlib/Probability/Process/Filtration.lean,Mathlib/RingTheory/Congruence/Basic.lean,Mathlib/RingTheory/Finiteness/Small.lean,Mathlib/RingTheory/NonUnitalSubring/Basic.lean,Mathlib/RingTheory/NonUnitalSubsemiring/Basic.lean,Mathlib/RingTheory/TwoSidedIdeal/Lattice.lean,Mathlib/RingTheory/UniqueFactorizationDomain/FactorSet.lean,Mathlib/RingTheory/Valuation/ValuationSubring.lean,Mathlib/Topology/Algebra/Group/GroupTopology.lean,Mathlib/Topology/Category/TopCat/OpenNhds.lean,Mathlib/Topology/LocallyFinsupp.lean,Mathlib/Topology/MetricSpace/BundledFun.lean,Mathlib/Topology/UniformSpace/Basic.lean |
82 |
14 |
['JovanGerb', 'bryangingechen', 'eric-wieser', 'github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'leanprover-community-mathlib4-bot'] |
nobody |
70-23476 2 months ago |
70-23476 2 months ago |
1-85670 1 day |
24710 |
chrisflav author:chrisflav |
chore(Data/Set): `tsum` version of `Set.encard_iUnion_of_finite` for non-finite types |
As requested here: https://github.com/leanprover-community/mathlib4/pull/23849#discussion_r2081070200
---
- [ ] depends on: #23849
[](https://gitpod.io/from-referrer/)
|
t-data
merge-conflict
|
163/0 |
Mathlib.lean,Mathlib/Algebra/BigOperators/Finprod.lean,Mathlib/Data/Set/Card/Arithmetic.lean,Mathlib/Data/Set/Card/InfiniteArithmetic.lean,Mathlib/Data/Set/Finite/Lattice.lean,Mathlib/Topology/Algebra/InfiniteSum/Order.lean,Mathlib/Topology/Instances/ENat/Lemmas.lean |
7 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
70-23474 2 months ago |
70-23474 2 months ago |
1-80465 1 day |
24823 |
eric-wieser author:eric-wieser |
refactor: add `hom` lemmas for the `MonoidalCategory` structure on `ModuleCat` |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
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 |
21 |
['101damnations', 'YaelDillies', 'eric-wieser', 'github-actions', 'joelriou', 'kbuzzard', 'leanprover-community-bot-assistant'] |
101damnations assignee:101damnations |
70-23473 2 months ago |
70-23473 2 months ago |
43-42841 43 days |
25071 |
erdOne author:erdOne |
feat(EllipticCurve): basic API for singular cubics |
---
[](https://gitpod.io/from-referrer/)
|
t-algebraic-geometry
merge-conflict
|
320/0 |
Mathlib.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Singular/Basic.lean,Mathlib/AlgebraicGeometry/EllipticCurve/VariableChange.lean |
3 |
35 |
['Multramate', 'acmepjz', 'erdOne', 'github-actions', 'leanprover-community-bot-assistant'] |
nobody |
70-23227 2 months ago |
70-23228 2 months ago |
45-4961 45 days |
25197 |
eric-wieser author:eric-wieser |
feat: Finset.sum induction for tensor products. |
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebra
merge-conflict
label:t-algebra$ |
81/0 |
Mathlib/LinearAlgebra/TensorProduct/Basic.lean |
1 |
2 |
['github-actions', 'leanprover-community-bot-assistant'] |
nobody |
70-23225 2 months ago |
70-23226 2 months ago |
0-0 0 seconds |
25218 |
kckennylau author:kckennylau |
feat(AlgebraicGeometry): Tate normal form of elliptic curves |
---
[](https://gitpod.io/from-referrer/)
|
awaiting-zulip
new-contributor
t-algebraic-geometry
merge-conflict
|
291/26 |
Mathlib.lean,Mathlib/AlgebraicGeometry/EllipticCurve/IsomOfJ.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Modular/TateNormalForm.lean,Mathlib/AlgebraicGeometry/EllipticCurve/NormalForms.lean,Mathlib/AlgebraicGeometry/EllipticCurve/VariableChange.lean |
5 |
31 |
['MichaelStollBayreuth', 'Multramate', 'acmepjz', 'github-actions', 'grunweg', 'kckennylau', 'leanprover-community-bot-assistant'] |
nobody |
70-23224 2 months ago |
70-23225 2 months ago |
6-51040 6 days |
25247 |
alreadydone author:alreadydone |
Projective contraction |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
label:t-algebra$ |
160/31 |
Mathlib/Data/Finsupp/Defs.lean,Mathlib/LinearAlgebra/Contraction.lean,Mathlib/LinearAlgebra/Pi.lean,Mathlib/RingTheory/Finiteness/Finsupp.lean |
4 |
2 |
['github-actions', 'leanprover-community-bot-assistant'] |
nobody |
70-23221 2 months ago |
70-23222 2 months ago |
0-30 30 seconds |
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
merge-conflict
label:t-algebra$ |
871/0 |
.vscode/settings.json,Mathlib.lean,Mathlib/RingTheory/EmbeddingDimension.lean,Mathlib/RingTheory/LocalRingDimension.lean,Mathlib/RingTheory/RegularLocalRing.lean |
5 |
6 |
['Brian-Nugent', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'yuanyi-350'] |
nobody |
70-23220 2 months ago |
70-23220 2 months ago |
11-84822 11 days |
25561 |
callesonne author:callesonne |
feat(Category/Grpd): define the bicategory of groupoids |
---
[](https://gitpod.io/from-referrer/)
|
t-category-theory
merge-conflict
awaiting-author
|
179/25 |
Mathlib.lean,Mathlib/AlgebraicTopology/FundamentalGroupoid/InducedMaps.lean,Mathlib/CategoryTheory/Bicategory/Functor/Pseudofunctor.lean,Mathlib/CategoryTheory/Bicategory/Functor/Strict.lean,Mathlib/CategoryTheory/Category/Cat.lean,Mathlib/CategoryTheory/Category/Grpd.lean |
6 |
6 |
['callesonne', 'github-actions', 'joelriou', 'leanprover-community-bot-assistant', 'robin-carlier'] |
nobody |
70-23209 2 months ago |
70-23210 2 months ago |
11-11653 11 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
merge-conflict
|
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 |
2 |
['github-actions', 'leanprover-community-bot-assistant'] |
nobody |
70-23208 2 months ago |
70-23209 2 months ago |
26-17604 26 days |
25622 |
eric-wieser author:eric-wieser |
refactor: overhaul instances on LocalizedModule |
This:
* Generalizes the `SMul`, `Module`, and `Algebra` instances via appropriate compatibility conditions
* Generalizes the `Mul` instance to the non-unital setting
* Fixes instances diamonds for the `Nat`- and `Int`-actions
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
label:t-algebra$ |
167/111 |
Mathlib/Algebra/Module/LocalizedModule/Basic.lean |
1 |
4 |
['erdOne', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant'] |
nobody |
70-23082 2 months ago |
70-23083 2 months ago |
25-53155 25 days |
25671 |
eric-wieser author:eric-wieser |
refactor: generalize `OreSet` to work for bimodules |
---
[](https://gitpod.io/from-referrer/)
|
large-import
merge-conflict
|
243/256 |
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 |
2 |
['github-actions', 'leanprover-community-bot-assistant'] |
nobody |
70-23080 2 months ago |
70-23081 2 months ago |
0-0 0 seconds |
25816 |
sgouezel author:sgouezel |
chore: kill coercion from EquivLike to Equiv |
---
[](https://gitpod.io/from-referrer/)
|
t-logic
merge-conflict
WIP
|
35/37 |
Mathlib/Logic/Equiv/Defs.lean |
1 |
2 |
['github-actions', 'leanprover-community-bot-assistant'] |
nobody |
70-23066 2 months ago |
70-23066 2 months ago |
0-1 1 second |
25887 |
eric-wieser author:eric-wieser |
feat: add `IsSMulTorsionFree` |
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebra
merge-conflict
label:t-algebra$ |
130/12 |
Mathlib/Algebra/Group/Action/TorsionFree.lean,Mathlib/Algebra/NoZeroSMulDivisors/Basic.lean,Mathlib/Algebra/Regular/Opposite.lean |
3 |
4 |
['YaelDillies', 'github-actions', 'leanprover-community-bot-assistant'] |
nobody |
70-22932 2 months ago |
70-22933 2 months ago |
0-0 0 seconds |
25901 |
callesonne author:callesonne |
feat(Bicategory/Opposites): add 1-cell opposite bicategory |
This PR adds the 1-cell opposite bicategory, where only the 1-morphisms are reversed.
---
[](https://gitpod.io/from-referrer/)
|
t-category-theory
merge-conflict
awaiting-author
|
219/1 |
Mathlib.lean,Mathlib/CategoryTheory/Bicategory/Opposites.lean,Mathlib/CategoryTheory/Opposites.lean,Mathlib/Tactic/CategoryTheory/Reassoc.lean |
4 |
10 |
['callesonne', 'github-actions', 'joelriou', 'leanprover-bot', 'leanprover-community-bot-assistant'] |
nobody |
70-22929 2 months ago |
70-22929 2 months ago |
0-14913 4 hours |
25963 |
artie2000 author:artie2000 |
refactor: Abstract out the substructure lattice construction and SetLike closure operators |
---
[](https://gitpod.io/from-referrer/)
Original PR: https://github.com/leanprover-community/mathlib4/pull/20836 |
merge-conflict |
354/179 |
Mathlib/Algebra/Group/Subsemigroup/Basic.lean,Mathlib/Algebra/Group/Subsemigroup/Defs.lean,Mathlib/Data/SetLike/Basic.lean,Mathlib/Data/SetLike/Closure.lean |
4 |
2 |
['github-actions', 'leanprover-community-bot-assistant'] |
nobody |
70-22917 2 months ago |
70-22918 2 months ago |
0-0 0 seconds |
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
merge-conflict
|
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 |
3 |
['Multramate', 'github-actions', 'leanprover-community-bot-assistant'] |
nobody |
70-22915 2 months ago |
70-22915 2 months ago |
18-21880 18 days |
26002 |
robin-carlier author:robin-carlier |
feat(CategoryTheory/Monoidal/Action): action of `Type` on categories with coproducts |
We show that if a category admits coproducts of size `w`, then `Type w` acts on the left on that category.
---
[](https://gitpod.io/from-referrer/)
|
t-category-theory
merge-conflict
WIP
|
213/0 |
Mathlib.lean,Mathlib/CategoryTheory/Monoidal/Action/ChosenTypeCopowers.lean |
2 |
2 |
['github-actions', 'leanprover-community-bot-assistant'] |
nobody |
70-22913 2 months ago |
70-22914 2 months ago |
0-0 0 seconds |
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
merge-conflict
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 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'linesthatinterlace'] |
nobody |
70-22911 2 months ago |
70-22912 2 months ago |
17-68825 17 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
merge-conflict
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 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'linesthatinterlace'] |
nobody |
70-22910 2 months ago |
70-22911 2 months ago |
17-68773 17 days |
26071 |
linesthatinterlace author:linesthatinterlace |
feat: Add `id` and `comp` classes for `FunLike` and `refl`, `trans` and `symm` classes for `EquivLike` |
Adds classes depending on `FunLike` that capture "this has an identity/this has a notion of composition".
---
This is a prototype and comments on this are requested. I think a similar model could be used to create a generalisation for Equiv.symm.
[](https://gitpod.io/from-referrer/)
|
t-data
RFC
merge-conflict
WIP
|
333/47 |
Mathlib/Data/FunLike/Basic.lean,Mathlib/Data/FunLike/Equiv.lean,Mathlib/Logic/Equiv/Defs.lean |
3 |
21 |
['Rob23oba', 'github-actions', 'leanprover-community-bot-assistant', 'linesthatinterlace'] |
nobody |
70-20927 2 months ago |
70-20928 2 months ago |
0-1 1 second |
26090 |
grunweg author:grunweg |
chore: make `finiteness` a default tactic |
Opening for discussion.
This PR continues the work from #25119. |
merge-conflict |
423/366 |
Archive/Wiedijk100Theorems/BallotProblem.lean,Mathlib/Analysis/Analytic/Uniqueness.lean,Mathlib/Analysis/Asymptotics/ExpGrowth.lean,Mathlib/Analysis/Calculus/ContDiff/Basic.lean,Mathlib/Analysis/Convex/Integral.lean,Mathlib/Analysis/Fourier/AddCircle.lean,Mathlib/Analysis/Fourier/AddCircleMulti.lean,Mathlib/Analysis/FunctionalSpaces/SobolevInequality.lean,Mathlib/Analysis/Normed/Field/Basic.lean,Mathlib/Analysis/Normed/Lp/PiLp.lean,Mathlib/Analysis/Normed/Lp/ProdLp.lean,Mathlib/Analysis/Normed/Lp/lpSpace.lean,Mathlib/Analysis/SpecialFunctions/Pow/Continuity.lean,Mathlib/Analysis/SpecialFunctions/Pow/NNReal.lean,Mathlib/Analysis/SpecificLimits/Basic.lean,Mathlib/Data/ENNReal/Basic.lean,Mathlib/Data/ENNReal/Holder.lean,Mathlib/Data/ENNReal/Inv.lean,Mathlib/Data/ENNReal/Operations.lean,Mathlib/Data/ENNReal/Real.lean,Mathlib/Data/EReal/Basic.lean,Mathlib/Data/EReal/Operations.lean,Mathlib/InformationTheory/KullbackLeibler/Basic.lean,Mathlib/MeasureTheory/Covering/Besicovitch.lean,Mathlib/MeasureTheory/Function/AEEqOfIntegral.lean,Mathlib/MeasureTheory/Function/ContinuousMapDense.lean,Mathlib/MeasureTheory/Function/ConvergenceInMeasure.lean,Mathlib/MeasureTheory/Function/Egorov.lean,Mathlib/MeasureTheory/Function/Jacobian.lean,Mathlib/MeasureTheory/Function/L1Space/AEEqFun.lean,Mathlib/MeasureTheory/Function/L2Space.lean,Mathlib/MeasureTheory/Function/LocallyIntegrable.lean,Mathlib/MeasureTheory/Function/LpSeminorm/Basic.lean,Mathlib/MeasureTheory/Function/LpSeminorm/ChebyshevMarkov.lean,Mathlib/MeasureTheory/Function/LpSeminorm/CompareExp.lean,Mathlib/MeasureTheory/Function/LpSeminorm/Defs.lean,Mathlib/MeasureTheory/Function/LpSpace/Basic.lean,Mathlib/MeasureTheory/Function/LpSpace/Complete.lean,Mathlib/MeasureTheory/Function/LpSpace/Indicator.lean,Mathlib/MeasureTheory/Function/SimpleFuncDenseLp.lean,Mathlib/MeasureTheory/Function/UniformIntegrable.lean,Mathlib/MeasureTheory/Integral/Bochner/Basic.lean,Mathlib/MeasureTheory/Integral/MeanInequalities.lean,Mathlib/MeasureTheory/Integral/Prod.lean,Mathlib/MeasureTheory/Integral/RieszMarkovKakutani/Real.lean,Mathlib/MeasureTheory/Measure/Decomposition/IntegralRNDeriv.lean,Mathlib/MeasureTheory/Measure/Decomposition/Lebesgue.lean,Mathlib/MeasureTheory/Measure/Haar/Basic.lean,Mathlib/MeasureTheory/Measure/Haar/DistribChar.lean,Mathlib/MeasureTheory/Measure/Haar/Quotient.lean,Mathlib/MeasureTheory/Measure/Haar/Unique.lean,Mathlib/MeasureTheory/Measure/Lebesgue/EqHaar.lean,Mathlib/MeasureTheory/Measure/LevyProkhorovMetric.lean,Mathlib/MeasureTheory/Measure/Real.lean,Mathlib/MeasureTheory/Measure/Restrict.lean,Mathlib/MeasureTheory/Measure/Tilted.lean,Mathlib/MeasureTheory/Measure/Typeclasses/Finite.lean,Mathlib/NumberTheory/NumberField/Discriminant/Basic.lean,Mathlib/Probability/BorelCantelli.lean,Mathlib/Probability/Independence/Conditional.lean,Mathlib/Probability/Integration.lean,Mathlib/Probability/Kernel/Composition/IntegralCompProd.lean,Mathlib/Probability/Kernel/Disintegration/CondCDF.lean,Mathlib/Probability/Kernel/Disintegration/Density.lean,Mathlib/Probability/Martingale/Convergence.lean,Mathlib/Probability/Martingale/OptionalStopping.lean,Mathlib/Probability/Moments/CovarianceBilin.lean,Mathlib/Probability/Moments/Tilted.lean,Mathlib/Probability/Moments/Variance.lean,Mathlib/Probability/UniformOn.lean,Mathlib/Topology/MetricSpace/Bounded.lean,Mathlib/Topology/MetricSpace/Perfect.lean,scripts/noshake.json |
73 |
3 |
['github-actions', 'grunweg', 'leanprover-community-bot-assistant'] |
nobody |
70-20925 2 months ago |
70-20926 2 months ago |
16-56825 16 days |
26178 |
ppls-nd-prs author:ppls-nd-prs |
feat(CategoryTheory/Limits): Fubini for products |
We show that the product of products is a product indexed by the sigma type.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-category-theory
merge-conflict
awaiting-author
|
17/0 |
Mathlib/CategoryTheory/Limits/Shapes/Products.lean |
1 |
5 |
['chrisflav', 'github-actions', 'leanprover-community-bot-assistant', 'ppls-nd-prs', 'robin-carlier'] |
robin-carlier assignee:robin-carlier |
70-20914 2 months ago |
70-20915 2 months ago |
0-47665 13 hours |
26384 |
jjdishere author:jjdishere |
feat(RingTheory/Perfectoid): Fontaine's theta map is surjective |
This PR continues the work from #22332.
Original PR: https://github.com/leanprover-community/mathlib4/pull/22332 |
t-algebra
t-number-theory
merge-conflict
WIP
label:t-algebra$ |
1109/15 |
Mathlib.lean,Mathlib/Algebra/Ring/Aut.lean,Mathlib/FieldTheory/Perfect.lean,Mathlib/RingTheory/AdicCompletion/Basic.lean,Mathlib/RingTheory/Ideal/Maps.lean,Mathlib/RingTheory/Ideal/Quotient/Defs.lean,Mathlib/RingTheory/Ideal/Quotient/PowTransition.lean,Mathlib/RingTheory/Perfection.lean,Mathlib/RingTheory/Perfectoid/BDeRham.lean,Mathlib/RingTheory/Perfectoid/FontaineTheta.lean,Mathlib/RingTheory/Perfectoid/Untilt.lean,Mathlib/RingTheory/WittVector/Basic.lean,Mathlib/RingTheory/WittVector/Complete.lean,Mathlib/RingTheory/WittVector/TeichmullerSeries.lean,docs/references.bib |
15 |
3 |
['github-actions', 'jjdishere', 'leanprover-community-bot-assistant'] |
nobody |
70-20779 2 months ago |
70-20779 2 months ago |
0-135 2 minutes |
26388 |
jjdishere author:jjdishere |
feat(RingTheory/Perfectoid): Fontaine's theta map and the de Rham period rings |
This PR continues the work from #21564.
Original PR: https://github.com/leanprover-community/mathlib4/pull/21564 |
t-algebra
t-number-theory
merge-conflict
label:t-algebra$ |
1026/15 |
Mathlib.lean,Mathlib/Algebra/Ring/Aut.lean,Mathlib/FieldTheory/Perfect.lean,Mathlib/RingTheory/AdicCompletion/Basic.lean,Mathlib/RingTheory/Ideal/Maps.lean,Mathlib/RingTheory/Ideal/Quotient/Defs.lean,Mathlib/RingTheory/Ideal/Quotient/PowTransition.lean,Mathlib/RingTheory/Perfection.lean,Mathlib/RingTheory/Perfectoid/BDeRham.lean,Mathlib/RingTheory/Perfectoid/FontaineTheta.lean,Mathlib/RingTheory/Perfectoid/Untilt.lean,Mathlib/RingTheory/WittVector/Basic.lean,Mathlib/RingTheory/WittVector/Complete.lean,Mathlib/RingTheory/WittVector/TeichmullerSeries.lean,docs/references.bib |
15 |
n/a |
['github-actions', 'jjdishere', 'leanprover-community-bot-assistant', 'riccardobrasca'] |
riccardobrasca assignee:riccardobrasca |
70-20777 2 months ago |
unknown |
unknown |
26436 |
AntoineChambert-Loir author:AntoineChambert-Loir |
feat(Mathlib/Data/Nat/Prime/Defs): fuel Nat.minFac |
This is a fueled version of docs#Nat.minFacAux that can now be checked by `decide`.
---
[](https://gitpod.io/from-referrer/)
|
t-data
merge-conflict
|
53/48 |
Mathlib/Data/Nat/Prime/Defs.lean |
1 |
2 |
['github-actions', 'leanprover-community-bot-assistant'] |
nobody |
70-20773 2 months ago |
70-20773 2 months ago |
8-58125 8 days |
26776 |
sgouezel author:sgouezel |
refactor: make `I` an outparam, and use forgetful inheritance in products |
I consider this as a failed experiment, so it's not for merging.
---
[](https://gitpod.io/from-referrer/)
|
RFC
merge-conflict
WIP
|
2411/1664 |
Mathlib/Analysis/Asymptotics/Defs.lean,Mathlib/Analysis/Asymptotics/Lemmas.lean,Mathlib/Analysis/CStarAlgebra/CStarMatrix.lean,Mathlib/Analysis/CStarAlgebra/Classes.lean,Mathlib/Analysis/CStarAlgebra/Module/Constructions.lean,Mathlib/Analysis/Calculus/InverseFunctionTheorem/ApproximatesLinearOn.lean,Mathlib/Analysis/Calculus/TangentCone.lean,Mathlib/Analysis/Calculus/TangentConeDef.lean,Mathlib/Analysis/Complex/Circle.lean,Mathlib/Analysis/Complex/UnitDisc/Basic.lean,Mathlib/Analysis/Complex/UpperHalfPlane/Topology.lean,Mathlib/Analysis/Normed/Module/Basic.lean,Mathlib/Analysis/Normed/Module/Prod.lean,Mathlib/Analysis/NormedSpace/HomeomorphBall.lean,Mathlib/Analysis/NormedSpace/Multilinear/Basic.lean,Mathlib/Analysis/NormedSpace/OperatorNorm/Basic.lean,Mathlib/Analysis/SpecialFunctions/Log/Basic.lean,Mathlib/Analysis/SpecialFunctions/PolarCoord.lean,Mathlib/Analysis/SpecialFunctions/Sqrt.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Arctan.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Inverse.lean,Mathlib/Geometry/Manifold/Algebra/Monoid.lean,Mathlib/Geometry/Manifold/AnalyticManifold.lean,Mathlib/Geometry/Manifold/ChartedSpace.lean,Mathlib/Geometry/Manifold/Complex.lean,Mathlib/Geometry/Manifold/ContMDiff/Basic.lean,Mathlib/Geometry/Manifold/ContMDiff/Constructions.lean,Mathlib/Geometry/Manifold/ContMDiff/Defs.lean,Mathlib/Geometry/Manifold/ContMDiff/NormedSpace.lean,Mathlib/Geometry/Manifold/Instances/Real.lean,Mathlib/Geometry/Manifold/Instances/Sphere.lean,Mathlib/Geometry/Manifold/IsManifold/Basic.lean,Mathlib/Geometry/Manifold/IsManifold/ExtChartAt.lean,Mathlib/Geometry/Manifold/IsManifold/ModelWithCornersDef.lean,Mathlib/Geometry/Manifold/LocalDiffeomorph.lean,Mathlib/Geometry/Manifold/LocalInvariantProperties.lean,Mathlib/Geometry/Manifold/MFDeriv/Atlas.lean,Mathlib/Geometry/Manifold/MFDeriv/Basic.lean,Mathlib/Geometry/Manifold/MFDeriv/Defs.lean,Mathlib/Geometry/Manifold/MFDeriv/FDeriv.lean,Mathlib/Geometry/Manifold/MFDeriv/SpecificFunctions.lean,Mathlib/Geometry/Manifold/MFDeriv/UniqueDifferential.lean,Mathlib/Geometry/Manifold/VectorBundle/Basic.lean,Mathlib/Geometry/Manifold/VectorBundle/FiberwiseLinear.lean,Mathlib/Geometry/Manifold/VectorBundle/Hom.lean,Mathlib/Geometry/Manifold/VectorBundle/MDifferentiable.lean,Mathlib/Geometry/Manifold/VectorBundle/Tangent.lean,Mathlib/MeasureTheory/Constructions/BorelSpace/Basic.lean,Mathlib/MeasureTheory/Function/SimpleFuncDenseLp.lean,Mathlib/NumberTheory/Modular.lean,Mathlib/NumberTheory/NumberField/CanonicalEmbedding/NormLeOne.lean,Mathlib/Topology/Algebra/Constructions.lean,Mathlib/Topology/Algebra/Module/LocallyConvex.lean,Mathlib/Topology/Algebra/PontryaginDual.lean,Mathlib/Topology/Bases.lean,Mathlib/Topology/Basic.lean,Mathlib/Topology/CWComplex/Classical/Basic.lean,Mathlib/Topology/Clopen.lean,Mathlib/Topology/Connected/TotallyDisconnected.lean,Mathlib/Topology/Constructions/SumProd.lean,Mathlib/Topology/ContinuousMap/Bounded/Basic.lean,Mathlib/Topology/ContinuousOn.lean,Mathlib/Topology/ContinuousOnMore.lean,Mathlib/Topology/Covering.lean,Mathlib/Topology/Defs/Basic.lean,Mathlib/Topology/Defs/Filter.lean,Mathlib/Topology/FiberBundle/Basic.lean,Mathlib/Topology/FiberBundle/Constructions.lean,Mathlib/Topology/FiberBundle/Trivialization.lean,Mathlib/Topology/Inseparable.lean,Mathlib/Topology/Instances/AddCircle.lean,Mathlib/Topology/Instances/Shrink.lean,Mathlib/Topology/Instances/TrivSqZeroExt.lean,Mathlib/Topology/Irreducible.lean,Mathlib/Topology/IsLocalHomeomorph.lean,Mathlib/Topology/LocallyFinite.lean,Mathlib/Topology/OmegaCompletePartialOrder.lean,Mathlib/Topology/Order/LeftRight.lean,Mathlib/Topology/PartialHomeomorph.lean,Mathlib/Topology/PartialHomeomorphMore.lean,Mathlib/Topology/Separation/Basic.lean,Mathlib/Topology/Separation/Regular.lean,Mathlib/Topology/UniformSpace/Basic.lean,Mathlib/Topology/UniformSpace/Cauchy.lean,Mathlib/Topology/UniformSpace/Defs.lean,Mathlib/Topology/UniformSpace/UniformConvergenceTopology.lean,Mathlib/Topology/VectorBundle/Basic.lean,Mathlib/Topology/VectorBundle/Hom.lean |
88 |
0 |
[] |
nobody |
70-10858 2 months ago |
70-10858 2 months ago |
0-1 1 second |
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
merge-conflict
|
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 |
18 |
['ADedecker', 'alreadydone', 'digama0', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'tb65536'] |
nobody |
69-61491 2 months ago |
69-61492 2 months ago |
73-67280 73 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
merge-conflict
|
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 |
2 |
['github-actions', 'leanprover-community-bot-assistant'] |
nobody |
68-74744 2 months ago |
68-74745 2 months ago |
69-52361 69 days |
26647 |
b-mehta author:b-mehta |
feat(Data/Sym/Sym2): lift commutative operations to sym2 |
While we have `Sym2.lift`, it's often useful to lift operations which are known to be commutative to the typeclass system. Indeed, the existing `Sym2.mul` witnesses this already. Thus, this PR can also be seen as generalising `Sym2.mul`.
---
[](https://gitpod.io/from-referrer/)
|
t-data
merge-conflict
WIP
|
48/28 |
Mathlib/Data/Sym/Sym2.lean,Mathlib/Data/Sym/Sym2/Finsupp.lean,Mathlib/LinearAlgebra/QuadraticForm/Basic.lean,Mathlib/LinearAlgebra/QuadraticForm/Basis.lean |
4 |
12 |
['b-mehta', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant'] |
nobody |
68-26505 2 months ago |
68-26506 2 months ago |
3-73380 3 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
merge-conflict
|
18/0 |
Mathlib/Topology/StoneCech.lean |
1 |
2 |
['github-actions', 'leanprover-community-bot-assistant'] |
nobody |
67-4293 2 months ago |
67-4293 2 months ago |
20-8582 20 days |
23990 |
robertmaxton42 author:robertmaxton42 |
feat (Types.Colimits): Quot is functorial and colimitEquivQuot is natural |
Add `Functor.quotFunctor` to parallel `Functor.sectionsFunctor`, witnessing that `Quot` is functorial; add `colimNatIsoQuotFunctor` to parallel `limNatIsoSectionsFunctor`, witnessing that `colimitEquivQuot` is natural in the diagram $F$.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-category-theory
merge-conflict
awaiting-author
|
33/0 |
Mathlib/CategoryTheory/Limits/Types/Colimits.lean |
1 |
5 |
['github-actions', 'joelriou', 'leanprover-community-bot-assistant', 'robertmaxton42'] |
nobody |
66-31036 2 months ago |
66-31037 2 months ago |
8-28043 8 days |
10541 |
Louddy author:Louddy |
feat(Algebra/SkewMonoidAlgebra/Basic): add SkewMonoidAlgebra |
# Skew Monoid algebras
This file presents a skewed version of `Mathlib.Algebra.MonoidAlgebra.Basic`.
## Definition
We define `SkewMonoidAlgebra k G := G →₀ k` attached with a skewed convolution product.
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`.
This will be used in a later PR to define skew polynomial rings.
Co-authored-by: María Inés de Frutos Fernández <[mariaines.dff@gmail.com](mailto:mariaines.dff@gmail.com)>
---
- [x] depends on: #15878
- [x] depends on: #19084
- [x] depends on: #22078
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-algebra
merge-conflict
WIP
label:t-algebra$ |
1624/0 |
Mathlib.lean,Mathlib/Algebra/Group/InjSurj.lean,Mathlib/Algebra/SkewMonoidAlgebra/Basic.lean,Mathlib/Algebra/SkewMonoidAlgebra/Lift.lean |
4 |
105 |
['AntoineChambert-Loir', 'Louddy', 'YaelDillies', 'eric-wieser', 'fpvandoorn', 'github-actions', 'mariainesdff', 'mathlib4-dependent-issues-bot', 'mattrobball'] |
AntoineChambert-Loir assignee:AntoineChambert-Loir |
65-78702 2 months ago |
65-78704 2 months ago |
179-12934 179 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
merge-conflict
|
48/24 |
Mathlib/Topology/Separation/Regular.lean,Mathlib/Topology/UniformSpace/OfCompactT2.lean |
2 |
4 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
65-66468 2 months ago |
65-66469 2 months ago |
76-65641 76 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
merge-conflict
|
920/0 |
Mathlib.lean,Mathlib/Topology/Compactification/OnePointHomeomorph.lean,Mathlib/Topology/Compactification/OnePointRealLemmas.lean |
3 |
3 |
['bjoernkjoshanssen', 'github-actions', 'leanprover-community-bot-assistant'] |
nobody |
65-10367 2 months ago |
67-4295 2 months ago |
21-20473 21 days |
24096 |
plp127 author:plp127 |
feat(Topology): Completely Regular Space iff Uniformizable |
Proves that `CompletelyRegularSpace`s are uniformizable and that `UniformSpace`s are completely regular.
---
- [x] depends on: #24179
- [x] depends on: #24173
[](https://gitpod.io/from-referrer/)
|
t-topology
merge-conflict
|
339/1 |
Mathlib.lean,Mathlib/Topology/Bases.lean,Mathlib/Topology/UniformSpace/Basic.lean,Mathlib/Topology/UniformSpace/Defs.lean,Mathlib/Topology/UniformSpace/Uniformizable.lean |
5 |
10 |
['alreadydone', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'plp127'] |
nobody |
63-63995 2 months ago |
64-23012 2 months ago |
2-8297 2 days |
25710 |
Paul-Lez author:Paul-Lez |
feat(Mathlib/Analysis/PDE/Quasilinear/Characteristics): the method of characteristics for first order quasilinear PDEs |
---
- [x] depends on: #25708
[](https://gitpod.io/from-referrer/)
|
t-analysis
merge-conflict
WIP
|
531/0 |
Mathlib/Analysis/Calculus/TangentCone.lean,Mathlib/Analysis/ODE/Gronwall.lean,Mathlib/Analysis/PDE/Quasilinear/Characteristics.lean,Mathlib/Topology/MetricSpace/Pseudo/Defs.lean,Mathlib/Topology/Separation/Basic.lean |
5 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
63-62188 2 months ago |
63-62189 2 months ago |
0-1343 22 minutes |
26966 |
vihdzp author:vihdzp |
feat: the Dedekind-MacNeille completion |
We define the type of Dedekind cuts `DedekindCut α` as an abbreviation for `Concept α α (· ≤ ·)`. We prove that it's the smallest complete lattice containing a given partial order, in the sense that any embedding from `α` into a complete lattice factors through it.
---
The idea here is that one should be able to work with Dedekind cuts without knowing what a concept lattice is; whence the abbreviation. See [Zulip](https://leanprover.zulipchat.com/#narrow/channel/116395-maths/topic/Dedekind-MacNeille.20completion.2E/near/528004148).
[](https://gitpod.io/from-referrer/)
|
t-order
merge-conflict
awaiting-author
|
133/1 |
Mathlib.lean,Mathlib/Order/Concept.lean,Mathlib/Order/Dedekind.lean |
3 |
11 |
['YaelDillies', 'github-actions', 'leanprover-community-bot-assistant', 'linesthatinterlace', 'vihdzp'] |
nobody |
63-61122 2 months ago |
63-61123 2 months ago |
0-0 0 seconds |
21039 |
eric-wieser author:eric-wieser |
hack: override `instance` to insert `fast_instance%` |
---
[](https://gitpod.io/from-referrer/)
|
t-meta
merge-conflict
please-adopt
|
40/4 |
Mathlib/Algebra/Equiv/TransferInstance.lean,Mathlib/RingTheory/Ideal/Maximal.lean,Mathlib/Tactic/FastInstance.lean,Mathlib/Topology/FiberBundle/Basic.lean |
4 |
2 |
['github-actions', 'leanprover-community-bot-assistant'] |
nobody |
63-53395 2 months ago |
63-53395 2 months ago |
0-0 0 seconds |
26911 |
JovanGerb author:JovanGerb |
chore: fix naming of `mono` and `monotone` |
The naming convention says:
"We use `_mono` for `a ≤ b → f a ≤ f b` and `_anti` for `a ≤ b → f b ≤ f a`, so we also use `_monotone` for `Monotone f`, `_antitone` for `Antitone f`, `_strictMono` for `StrictMono f`, `_strictAnti` for `StrictAnti f`, etc..."
This PR swaps `mono`/`anti` and `monotone`/`antitone` where required so that `monotone` refers to `Monotone`, while `mono` refers to a lemma that might be tagged with `@[gcongr]`
This PR does not address
- `mul_left_monotone` and `mul_right_monotone` are exactly the wrong way around
- `monotone_right`/`mono_right` vs `right_monotone`/`right_mono`
- `monotone_arcsin` vs `arcsin_monotone`
edit: TODO: `ideal_mono` and friends
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict
delegated
|
238/171 |
Archive/Imo/Imo1962Q1.lean,Archive/Wiedijk100Theorems/AbelRuffini.lean,Archive/Wiedijk100Theorems/SumOfPrimeReciprocalsDiverges.lean,Counterexamples/DiscreteTopologyNonDiscreteUniformity.lean,Mathlib/Algebra/Group/Pointwise/Finset/Basic.lean,Mathlib/Algebra/Group/Pointwise/Set/Basic.lean,Mathlib/Algebra/Order/Field/Basic.lean,Mathlib/Algebra/Order/Group/Basic.lean,Mathlib/Algebra/Order/Group/Finset.lean,Mathlib/Algebra/Order/Group/PosPart.lean,Mathlib/Algebra/Order/GroupWithZero/Unbundled/Basic.lean,Mathlib/Algebra/Order/Monoid/Unbundled/Basic.lean,Mathlib/Algebra/Order/Monoid/Unbundled/Pow.lean,Mathlib/Algebra/Order/ToIntervalMod.lean,Mathlib/Algebra/Polynomial/Degree/CardPowDegree.lean,Mathlib/AlgebraicGeometry/IdealSheaf/Basic.lean,Mathlib/Analysis/Analytic/Composition.lean,Mathlib/Analysis/Convex/Deriv.lean,Mathlib/Analysis/Normed/Order/UpperLower.lean,Mathlib/Analysis/PSeries.lean,Mathlib/Analysis/SpecialFunctions/Pow/Continuity.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Basic.lean,Mathlib/Analysis/SpecificLimits/Basic.lean,Mathlib/Analysis/SpecificLimits/FloorPow.lean,Mathlib/Combinatorics/SetFamily/Kleitman.lean,Mathlib/Combinatorics/SimpleGraph/Girth.lean,Mathlib/Combinatorics/SimpleGraph/Regularity/Chunk.lean,Mathlib/Combinatorics/SimpleGraph/Regularity/Lemma.lean,Mathlib/Computability/Ackermann.lean,Mathlib/Data/ENNReal/Inv.lean,Mathlib/Data/ENNReal/Operations.lean,Mathlib/Data/Nat/Choose/Factorization.lean,Mathlib/Data/Real/Pi/Bounds.lean,Mathlib/LinearAlgebra/AffineSpace/AffineMap.lean,Mathlib/MeasureTheory/Constructions/BorelSpace/Basic.lean,Mathlib/MeasureTheory/Constructions/Polish/Basic.lean,Mathlib/MeasureTheory/MeasurableSpace/MeasurablyGenerated.lean,Mathlib/MeasureTheory/OuterMeasure/Operations.lean,Mathlib/NumberTheory/Bertrand.lean,Mathlib/NumberTheory/FermatPsp.lean,Mathlib/NumberTheory/Padics/Hensel.lean,Mathlib/Order/Concept.lean,Mathlib/Order/Filter/AtTopBot/Defs.lean,Mathlib/Order/Fin/Basic.lean,Mathlib/Order/Heyting/Basic.lean,Mathlib/Order/Heyting/Boundary.lean,Mathlib/Order/Heyting/Regular.lean,Mathlib/Order/Hom/Set.lean,Mathlib/Order/Interval/Set/Fin.lean,Mathlib/Order/KrullDimension.lean,Mathlib/Order/UpperLower/Closure.lean,Mathlib/Probability/StrongLaw.lean,Mathlib/RingTheory/DedekindDomain/Different.lean,Mathlib/RingTheory/DedekindDomain/Ideal.lean,Mathlib/RingTheory/FractionalIdeal/Basic.lean,Mathlib/RingTheory/FractionalIdeal/Operations.lean,Mathlib/Topology/EMetricSpace/Lipschitz.lean,Mathlib/Topology/MetricSpace/Antilipschitz.lean,Mathlib/Topology/MetricSpace/Holder.lean |
59 |
8 |
['JovanGerb', 'bryangingechen', 'github-actions', 'leanprover-community-bot-assistant', 'linesthatinterlace', 'mathlib-bors'] |
bryangingechen assignee:bryangingechen |
63-32100 2 months ago |
63-61124 2 months ago |
2-60107 2 days |
21838 |
joneugster author:joneugster |
feat(Cache): Allow arguments of the form `Mathlib.Data` which correspond to a folder but not a file |
---
- [x] depends on: #21834
[](https://gitpod.io/from-referrer/)
|
CI
t-meta
merge-conflict
awaiting-author
|
34/11 |
Cache/IO.lean,Cache/Main.lean |
2 |
11 |
['eric-wieser', 'github-actions', 'joneugster', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mergify'] |
nobody |
61-54252 1 month ago |
61-54253 1 month ago |
50-67617 50 days |
25611 |
erdOne author:erdOne |
chore(RingTheory): add `Algebra (FractionRing R) (FractionRing S)` |
Co-authored-by: Yakov Pechersky
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
label:t-algebra$ |
152/108 |
Mathlib.lean,Mathlib/Algebra/Algebra/NonZeroDivisors.lean,Mathlib/NumberTheory/RamificationInertia/Galois.lean,Mathlib/RingTheory/DedekindDomain/Different.lean,Mathlib/RingTheory/DedekindDomain/IntegralClosure.lean,Mathlib/RingTheory/Ideal/Norm/RelNorm.lean,Mathlib/RingTheory/IntegralClosure/IntegralRestrict.lean,Mathlib/RingTheory/Localization/FractionRing.lean,Mathlib/RingTheory/Localization/FractionRingAlgebra.lean,Mathlib/RingTheory/Localization/Integral.lean |
10 |
20 |
['alreadydone', 'erdOne', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'pechersky'] |
nobody |
59-79511 1 month ago |
59-79512 1 month ago |
36-35321 36 days |
27310 |
ADedecker author:ADedecker |
chore: semilinearize LinearAlgebra.TensorProduct.Basic |
This PR continues the work from #24208.
Original PR: https://github.com/leanprover-community/mathlib4/pull/24208 |
t-algebra
merge-conflict
label:t-algebra$ |
191/138 |
Mathlib/Algebra/Category/ModuleCat/ChangeOfRings.lean,Mathlib/Algebra/Category/ModuleCat/Monoidal/Closed.lean,Mathlib/Algebra/Lie/TensorProduct.lean,Mathlib/Algebra/Module/Equiv/Defs.lean,Mathlib/LinearAlgebra/BilinearForm/TensorProduct.lean,Mathlib/LinearAlgebra/BilinearMap.lean,Mathlib/LinearAlgebra/Dual/Lemmas.lean,Mathlib/LinearAlgebra/TensorPower/Basic.lean,Mathlib/LinearAlgebra/TensorProduct/Associator.lean,Mathlib/LinearAlgebra/TensorProduct/Basic.lean,Mathlib/LinearAlgebra/TensorProduct/Tower.lean,Mathlib/RingTheory/Coalgebra/Hom.lean |
12 |
0 |
[] |
nobody |
54-67109 1 month ago |
54-67109 1 month ago |
0-49 49 seconds |
25284 |
alreadydone author:alreadydone |
feat(LinearAlgebra/Contraction): bijectivity of `dualTensorHom` + generalize to CommSemiring |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
awaiting-author
label:t-algebra$ |
167/32 |
Mathlib/Data/Finsupp/Defs.lean,Mathlib/LinearAlgebra/Contraction.lean,Mathlib/LinearAlgebra/Pi.lean,Mathlib/LinearAlgebra/Trace.lean,Mathlib/RingTheory/Finiteness/Finsupp.lean |
5 |
16 |
['alreadydone', 'eric-wieser', 'github-actions', 'kckennylau', 'leanprover-bot', 'leanprover-community-bot-assistant'] |
nobody |
52-44051 1 month ago |
52-44051 1 month ago |
47-45899 47 days |
22749 |
joelriou author:joelriou |
feat(CategoryTheory/Abelian): the Gabriel-Popescu theorem as a localization with respect to a Serre class |
This PR introduces a structure `GabrielPopescuPackage C` which contains the information to say that the abelian category `C` is a localization of a category of modules with respect to a suitable Serre class.
---
- [x] depends on: #26033
- [ ] depends on: #26663
- [x] depends on: #22733
[](https://gitpod.io/from-referrer/)
|
t-category-theory
merge-conflict
WIP
|
202/6 |
Mathlib.lean,Mathlib/CategoryTheory/Abelian/GrothendieckCategory/ModuleEmbedding/GabrielPopescu.lean,Mathlib/CategoryTheory/Abelian/SerreClass/Bousfield.lean,Mathlib/CategoryTheory/Abelian/SerreClass/MorphismProperty.lean,Mathlib/CategoryTheory/ObjectProperty/ContainsZero.lean |
5 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
52-937 1 month ago |
52-939 1 month ago |
0-10930 3 hours |
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
merge-conflict
delegated
|
368/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 |
23 |
['chrisflav', 'erdOne', 'github-actions', 'jcommelin', 'leanprover-community-bot-assistant', 'mathlib-bors'] |
nobody |
51-80859 1 month ago |
51-80860 1 month ago |
17-3559 17 days |
26784 |
eric-wieser author:eric-wieser |
chore: remove suppress_compilation |
Still not exhaustive.
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict |
0/37 |
Mathlib/Algebra/Category/CoalgCat/ComonEquivalence.lean,Mathlib/Algebra/Category/ModuleCat/ChangeOfRings.lean,Mathlib/Algebra/Category/Ring/Constructions.lean,Mathlib/Algebra/Colimit/DirectLimit.lean,Mathlib/Algebra/Colimit/Module.lean,Mathlib/Algebra/Colimit/Ring.lean,Mathlib/AlgebraicGeometry/Limits.lean,Mathlib/Analysis/Normed/Algebra/Unitization.lean,Mathlib/Analysis/NormedSpace/Multilinear/Basic.lean,Mathlib/Analysis/NormedSpace/Multilinear/Curry.lean,Mathlib/Analysis/NormedSpace/OperatorNorm/Basic.lean,Mathlib/Analysis/NormedSpace/OperatorNorm/Bilinear.lean,Mathlib/Analysis/NormedSpace/OperatorNorm/Completeness.lean,Mathlib/Analysis/NormedSpace/OperatorNorm/Mul.lean,Mathlib/Analysis/NormedSpace/OperatorNorm/NNNorm.lean,Mathlib/Analysis/NormedSpace/OperatorNorm/NormedSpace.lean,Mathlib/CategoryTheory/Abelian/Projective/Resolution.lean,Mathlib/CategoryTheory/Monoidal/Internal/Module.lean |
18 |
2 |
['github-actions', 'leanprover-community-bot-assistant'] |
nobody |
51-59598 1 month ago |
51-59599 1 month ago |
0-0 0 seconds |
26804 |
kckennylau author:kckennylau |
(WIP) feat(SetTheory): ZFSet is a model of ZFC |
---
Depends on:
* [ ] #26644
`Mathlib/SetTheory/ZFC/Model.lean` is the main file, and it starts at Line 346.
[](https://gitpod.io/from-referrer/)
|
t-set-theory
merge-conflict
WIP
|
1245/0 |
Mathlib.lean,Mathlib/SetTheory/ZFC/Axioms.lean,Mathlib/SetTheory/ZFC/Model.lean,docs/references.bib |
4 |
2 |
['github-actions', 'leanprover-community-bot-assistant'] |
nobody |
51-11056 1 month ago |
51-11057 1 month ago |
0-163 2 minutes |
20428 |
madvorak author:madvorak |
feat(Data/Sign): lemmas about `∈ Set.range SignType.cast` |
---
Perhaps `in_set_range_singType_cast_iff_abs` needs to be moved somewhere downstream. |
t-data
merge-conflict
WIP
|
40/0 |
Mathlib/Data/Sign.lean |
1 |
10 |
['eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'madvorak'] |
nobody |
51-3549 1 month ago |
51-3550 1 month ago |
0-0 0 seconds |
23528 |
Ruben-VandeVelde author:Ruben-VandeVelde |
feat: add isOpen_setOf_affineIndependent |
From sphere-eversion.
---
[](https://gitpod.io/from-referrer/)
|
t-analysis
merge-conflict
delegated
|
15/0 |
Mathlib/Analysis/Normed/Module/FiniteDimension.lean |
1 |
5 |
['github-actions', 'grunweg', 'leanprover-community-bot-assistant', 'mathlib-bors', 'urkud'] |
nobody |
50-63603 1 month ago |
50-63604 1 month ago |
26-70139 26 days |
26608 |
vihdzp author:vihdzp |
feat(SetTheory/Cardinal/Aleph): `o.card ≤ ℵ_ o` and variants |
---
[](https://gitpod.io/from-referrer/)
|
t-set-theory
merge-conflict
|
24/0 |
Mathlib/SetTheory/Cardinal/Aleph.lean |
1 |
3 |
['github-actions', 'kckennylau', 'leanprover-community-bot-assistant'] |
nobody |
49-53968 1 month ago |
49-53969 1 month ago |
23-63406 23 days |
20029 |
FrederickPu author:FrederickPu |
Allow for Config attributes to be set directly |
Allow for Config attributes to be set directly when using initialize_simp_projection as per issue #19895
Basically modified initialize_simp_projection so that the user has the option of specifying a tuple of config option values.
Ex:
```
initialize_simp_projection MulEquiv (toFun → apply, invFun → symm_apply) (fullyApplied := false)
```
These config options are then converted into projections.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-meta
merge-conflict
WIP
|
34/4 |
Mathlib/Tactic/Simps/Basic.lean |
1 |
11 |
['FrederickPu', 'YaelDillies', 'fpvandoorn', 'github-actions', 'leanprover-community-bot-assistant'] |
nobody |
49-50649 1 month ago |
49-50650 1 month ago |
0-34081 9 hours |
13973 |
digama0 author:digama0 |
feat: lake exe refactor, initial framework |
This is the initial framework code for `lake exe refactor`. To use it, you add your refactoring to `Refactor/Main.lean` (note, you have to actually write some metaprogramming code here for the refactoring itself), and the harness will run it on specified files and apply the generated edits.
---
[](https://gitpod.io/from-referrer/)
|
t-meta
merge-conflict
awaiting-author
|
139/0 |
Refactor/Main.lean,lakefile.lean |
2 |
11 |
['adomani', 'digama0', 'eric-wieser', 'github-actions', 'joneugster', 'leanprover-community-bot-assistant', 'mattrobball'] |
nobody |
45-71510 1 month ago |
45-71511 1 month ago |
4-80741 4 days |
22092 |
fpvandoorn author:fpvandoorn |
perf: lower gcongr priority in group mono lemmas |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
WIP
label:t-algebra$ |
13/9 |
Mathlib/Algebra/Order/Monoid/Unbundled/Basic.lean |
1 |
6 |
['fpvandoorn', 'github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'leanprover-community-mathlib4-bot'] |
nobody |
43-85523 1 month ago |
43-85524 1 month ago |
0-6118 1 hour |
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
merge-conflict
|
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 |
11 |
['EtienneC30', 'b-mehta', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant'] |
nobody |
43-82396 1 month ago |
43-82396 1 month ago |
5-313 5 days |
12181 |
adomani author:adomani |
lint also `let` vs `have` |
This PR is symmetrical to #12157: here we lint for non-`Type`-valued `let`s.
---
[](https://gitpod.io/from-referrer/)
|
t-linter
merge-conflict
|
797/544 |
Archive/Imo/Imo1962Q1.lean,Archive/Wiedijk100Theorems/CubingACube.lean,Archive/Wiedijk100Theorems/FriendshipGraphs.lean,Mathlib.lean,Mathlib/Algebra/Algebra/Tower.lean,Mathlib/Algebra/BigOperators/Basic.lean,Mathlib/Algebra/DirectLimit.lean,Mathlib/Algebra/Group/UniqueProds.lean,Mathlib/Algebra/Homology/HomologicalComplexBiprod.lean,Mathlib/Algebra/Homology/HomologySequence.lean,Mathlib/Algebra/Homology/HomotopyCategory/Pretriangulated.lean,Mathlib/Algebra/Homology/Localization.lean,Mathlib/Algebra/Homology/ShortComplex/Abelian.lean,Mathlib/Algebra/Homology/ShortComplex/ConcreteCategory.lean,Mathlib/Algebra/Homology/ShortComplex/Exact.lean,Mathlib/Algebra/Homology/ShortComplex/ExactFunctor.lean,Mathlib/Algebra/Homology/ShortComplex/Homology.lean,Mathlib/Algebra/Homology/ShortComplex/LeftHomology.lean,Mathlib/Algebra/Homology/ShortComplex/Linear.lean,Mathlib/Algebra/Homology/ShortComplex/Preadditive.lean,Mathlib/Algebra/Homology/ShortComplex/PreservesHomology.lean,Mathlib/Algebra/Homology/ShortComplex/QuasiIso.lean,Mathlib/Algebra/Homology/ShortComplex/RightHomology.lean,Mathlib/Algebra/Lie/Engel.lean,Mathlib/Algebra/Lie/Killing.lean,Mathlib/Algebra/Module/PID.lean,Mathlib/Algebra/Module/Submodule/Localization.lean,Mathlib/Algebra/Module/Zlattice.lean,Mathlib/Algebra/MonoidAlgebra/Grading.lean,Mathlib/Algebra/MvPolynomial/Equiv.lean,Mathlib/Algebra/Order/CauSeq/Basic.lean,Mathlib/Algebra/Polynomial/FieldDivision.lean,Mathlib/Algebra/Polynomial/RingDivision.lean,Mathlib/AlgebraicGeometry/Morphisms/QuasiCompact.lean,Mathlib/AlgebraicGeometry/Morphisms/QuasiSeparated.lean,Mathlib/AlgebraicGeometry/ProjectiveSpectrum/Scheme.lean,Mathlib/AlgebraicGeometry/Pullbacks.lean,Mathlib/AlgebraicGeometry/StructureSheaf.lean,Mathlib/AlgebraicTopology/DoldKan/Homotopies.lean,Mathlib/Analysis/Calculus/ContDiff/Basic.lean,Mathlib/Analysis/Calculus/ContDiff/Bounds.lean,Mathlib/Analysis/Calculus/FDeriv/Comp.lean,Mathlib/Analysis/Calculus/Rademacher.lean,Mathlib/Analysis/Complex/Tietze.lean,Mathlib/Analysis/Convex/Between.lean,Mathlib/Analysis/Convolution.lean,Mathlib/Analysis/Fourier/RiemannLebesgueLemma.lean,Mathlib/Analysis/InnerProductSpace/GramSchmidtOrtho.lean,Mathlib/Analysis/InnerProductSpace/PiL2.lean,Mathlib/Analysis/InnerProductSpace/Rayleigh.lean,Mathlib/Analysis/NormedSpace/ContinuousAffineMap.lean,Mathlib/Analysis/NormedSpace/OperatorNorm/Completeness.lean,Mathlib/Analysis/NormedSpace/Spectrum.lean,Mathlib/Analysis/SpecialFunctions/Integrals.lean,Mathlib/CategoryTheory/Abelian/Basic.lean,Mathlib/CategoryTheory/Abelian/Exact.lean,Mathlib/CategoryTheory/Abelian/Pseudoelements.lean,Mathlib/CategoryTheory/Abelian/Transfer.lean,Mathlib/CategoryTheory/Adhesive.lean,Mathlib/CategoryTheory/Closed/Cartesian.lean,Mathlib/CategoryTheory/Closed/Monoidal.lean,Mathlib/CategoryTheory/Comma/Arrow.lean,Mathlib/CategoryTheory/EffectiveEpi/Extensive.lean,Mathlib/CategoryTheory/Extensive.lean,Mathlib/CategoryTheory/Functor/EpiMono.lean,Mathlib/CategoryTheory/Functor/KanExtension/Basic.lean,Mathlib/CategoryTheory/Galois/Basic.lean,Mathlib/CategoryTheory/Galois/Decomposition.lean,Mathlib/CategoryTheory/Galois/Examples.lean,Mathlib/CategoryTheory/GradedObject/Trifunctor.lean,Mathlib/CategoryTheory/IsConnected.lean,Mathlib/CategoryTheory/Limits/ConcreteCategory.lean,Mathlib/CategoryTheory/Limits/Constructions/EpiMono.lean,Mathlib/CategoryTheory/Limits/Constructions/WeaklyInitial.lean,Mathlib/CategoryTheory/Limits/FilteredColimitCommutesFiniteLimit.lean,Mathlib/CategoryTheory/Limits/Final.lean,Mathlib/CategoryTheory/Limits/FintypeCat.lean,Mathlib/CategoryTheory/Limits/Fubini.lean,Mathlib/CategoryTheory/Limits/IsLimit.lean,Mathlib/CategoryTheory/Limits/Preserves/Basic.lean,Mathlib/CategoryTheory/Limits/Shapes/FiniteLimits.lean,Mathlib/CategoryTheory/Limits/VanKampen.lean,Mathlib/CategoryTheory/Localization/LocalizerMorphism.lean,Mathlib/CategoryTheory/Localization/Pi.lean,Mathlib/CategoryTheory/Localization/Resolution.lean,Mathlib/CategoryTheory/Monad/Monadicity.lean,Mathlib/CategoryTheory/PUnit.lean,Mathlib/CategoryTheory/Sites/Coherent/CoherentSheaves.lean,Mathlib/CategoryTheory/Sites/Coherent/RegularSheaves.lean,Mathlib/CategoryTheory/Sites/Coverage.lean,Mathlib/CategoryTheory/Sites/LeftExact.lean,Mathlib/CategoryTheory/Sites/Preserves.lean,Mathlib/CategoryTheory/Sites/Pullback.lean,Mathlib/CategoryTheory/Sites/Sheaf.lean,Mathlib/CategoryTheory/Triangulated/Pretriangulated.lean,Mathlib/Combinatorics/Colex.lean,Mathlib/Combinatorics/SetFamily/Kleitman.lean,Mathlib/Combinatorics/SimpleGraph/Clique.lean,Mathlib/Combinatorics/SimpleGraph/Coloring.lean,Mathlib/Combinatorics/SimpleGraph/Connectivity.lean |
271 |
0 |
[] |
nobody |
43-81826 1 month ago |
43-81826 1 month ago |
0-0 0 seconds |
11021 |
jstoobysmith author:jstoobysmith |
feat(AlgebraicTopology) : add join of augmented SSets |
This pull-request adds the definition of the join of augmented SSets defined as contravariant functors from `WithInitial SimplexCategory` to `Type u`. In addition it shows that the join of two standard augmented SSets is again an augmented SSets.
From this the definition of the join of simplicial sets should follow easily.
To aid the above theory, an api for `WithInitial SimplexCategory` has been created, with the notion of the `join` and `split` (forming a sort of inverse to join) of objects in this category are defined.
---
[](https://gitpod.io/from-referrer/)
|
t-algebraic-topology
new-contributor
merge-conflict
WIP
|
2137/1 |
.gitignore,Mathlib.lean,Mathlib/AlgebraicTopology/Join.lean,Mathlib/AlgebraicTopology/SimplexCategory.lean,Mathlib/AlgebraicTopology/SimplexCategoryWithInitial.lean,Mathlib/AlgebraicTopology/SimplicialSet.lean |
6 |
47 |
['github-actions', 'jcommelin'] |
nobody |
43-81808 1 month ago |
43-81808 1 month ago |
1-20125 1 day |
10190 |
jstoobysmith author:jstoobysmith |
feat(AlgebraicTopology): add Augmented Simplex Category |
- Added the definition of the category FinLinOrd of finite linear ordered sets.
- Added the definition of the augmented simplex category `AugmentedSimplexCategory`, and showed it is the Skeleton of FinLinOrd.
- Showed that the category of augmented simplicial objects defined as a comma category is equivalent to the category of functors from `AugmentedSimplexCategory^\op`
---
[](https://gitpod.io/from-referrer/)
|
t-algebraic-topology
new-contributor
t-category-theory
merge-conflict
WIP
|
720/0 |
Mathlib.lean,Mathlib/AlgebraicTopology/AugmentedSimplexCategory.lean,Mathlib/AlgebraicTopology/SimplicialObject.lean,Mathlib/Order/Category/FinLinOrd.lean |
4 |
5 |
['TwoFX', 'YaelDillies', 'joelriou', 'jstoobysmith'] |
nobody |
43-81764 1 month ago |
43-81764 1 month ago |
7-63215 7 days |
10084 |
alreadydone author:alreadydone |
draft for Van Kampen |
The part about the homotopy lifting property for covering maps has been extracted to #22649
---
[](https://gitpod.io/from-referrer/)
|
t-algebraic-topology
merge-conflict
WIP
|
91/24 |
Mathlib/AlgebraicTopology/FundamentalGroupoid/Basic.lean,Mathlib/AlgebraicTopology/FundamentalGroupoid/VanKampen.lean |
2 |
1 |
['leanprover-community-bot-assistant'] |
nobody |
43-81673 1 month ago |
43-81673 1 month ago |
0-0 0 seconds |
26303 |
joelriou author:joelriou |
feat(AlgebraicTopology): the fundamental lemma of homotopical algebra |
Given a model category `C`, the fundamental lemma of homotopical algebra (Quillen) shows that it is possible to compute morphisms in the homotopy category of `C` (the localized category with respect to weak equivalences) from `X` to `Y` as a quotient of the type of morphisms from `X` to `Y` in `C` modulo an homotopy relation, when `X` is cofibrant and `Y` is fibrant. In particular, we obtain a version of the Whitehead theorem: a weak equivalence between bifibrant objects (both cofibrant and fibrant) is a homotopy equivalence. We also show that we obtain equivalent categories if we localize `C` or various fullsubcategories (cofibrant objetss, fibrant objects, bifibrant objects) with respect to weak equivalences. (This improves the first formalization I made in 2022 in Lean 3.)
(This is sorry-free, but still WIP. In order to do clean proofs, we shall also need the refactor of fullsubcategories...)
---
- [x] depends on: #26171
- [x] depends on: #26166
- [x] depends on: #26365
[](https://gitpod.io/from-referrer/)
|
t-algebraic-topology
large-import
t-category-theory
merge-conflict
WIP
|
3174/31 |
Mathlib.lean,Mathlib/AlgebraicTopology/ModelCategory/Basic.lean,Mathlib/AlgebraicTopology/ModelCategory/Bifibrant.lean,Mathlib/AlgebraicTopology/ModelCategory/BrownLemma.lean,Mathlib/AlgebraicTopology/ModelCategory/CategoryWithCofibrations.lean,Mathlib/AlgebraicTopology/ModelCategory/Cylinder.lean,Mathlib/AlgebraicTopology/ModelCategory/DerivabilityStructure.lean,Mathlib/AlgebraicTopology/ModelCategory/FundamentalLemma1.lean,Mathlib/AlgebraicTopology/ModelCategory/FundamentalLemma2.lean,Mathlib/AlgebraicTopology/ModelCategory/FundamentalLemma3.lean,Mathlib/AlgebraicTopology/ModelCategory/Homotopy.lean,Mathlib/AlgebraicTopology/ModelCategory/Instances.lean,Mathlib/AlgebraicTopology/ModelCategory/IsCofibrant.lean,Mathlib/AlgebraicTopology/ModelCategory/PathObject.lean,Mathlib/CategoryTheory/Localization/CalculusOfFractions/OfAdjunction.lean,Mathlib/CategoryTheory/Localization/Opposite.lean,Mathlib/CategoryTheory/Localization/Predicate.lean,Mathlib/CategoryTheory/Localization/Quotient.lean,Mathlib/CategoryTheory/MorphismProperty/Quotient.lean |
19 |
n/a |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
43-81599 1 month ago |
unknown |
unknown |
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/)
|
t-algebraic-topology
infinity-cosmos
t-meta
merge-conflict
|
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 |
23 |
['eric-wieser', 'gio256', 'github-actions', 'kim-em', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
eric-wieser assignee:eric-wieser |
43-81570 1 month ago |
43-81570 1 month ago |
88-84229 88 days |
26926 |
adomani author:adomani |
draft: `commandStart` more |
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-linter
merge-conflict
awaiting-author
WIP
|
3160/1085 |
Mathlib/Algebra/Category/ModuleCat/ChangeOfRings.lean,Mathlib/Algebra/Category/MonCat/Adjunctions.lean,Mathlib/Algebra/Divisibility/Basic.lean,Mathlib/Algebra/EuclideanDomain/Basic.lean,Mathlib/Algebra/Group/Commute/Defs.lean,Mathlib/Algebra/Group/Commute/Units.lean,Mathlib/Algebra/Group/Hom/CompTypeclasses.lean,Mathlib/Algebra/Group/Pointwise/Finset/Basic.lean,Mathlib/Algebra/Group/Semiconj/Basic.lean,Mathlib/Algebra/Group/Semiconj/Units.lean,Mathlib/Algebra/Group/UniqueProds/Basic.lean,Mathlib/Algebra/Homology/ComplexShape.lean,Mathlib/Algebra/Homology/Embedding/Boundary.lean,Mathlib/Algebra/Homology/HomotopyCategory/HomComplex.lean,Mathlib/Algebra/Homology/HomotopyCategory/HomComplexShift.lean,Mathlib/Algebra/Lie/LieTheorem.lean,Mathlib/Algebra/MvPolynomial/Equiv.lean,Mathlib/Algebra/Notation/Defs.lean,Mathlib/Algebra/Notation/Lemmas.lean,Mathlib/Algebra/Notation/Pi.lean,Mathlib/Algebra/Order/Antidiag/Pi.lean,Mathlib/Algebra/Order/Field/Basic.lean,Mathlib/Algebra/Polynomial/AlgebraMap.lean,Mathlib/Algebra/Polynomial/CoeffList.lean,Mathlib/Algebra/Polynomial/FieldDivision.lean,Mathlib/Algebra/Polynomial/Laurent.lean,Mathlib/Algebra/Polynomial/Sequence.lean,Mathlib/Algebra/Polynomial/Smeval.lean,Mathlib/Algebra/Quaternion.lean,Mathlib/Algebra/Ring/Ext.lean,Mathlib/AlgebraicTopology/DoldKan/Degeneracies.lean,Mathlib/AlgebraicTopology/DoldKan/FunctorGamma.lean,Mathlib/AlgebraicTopology/DoldKan/Homotopies.lean,Mathlib/AlgebraicTopology/DoldKan/HomotopyEquivalence.lean,Mathlib/AlgebraicTopology/DoldKan/NCompGamma.lean,Mathlib/AlgebraicTopology/DoldKan/Normalized.lean,Mathlib/AlgebraicTopology/DoldKan/Projections.lean,Mathlib/AlgebraicTopology/DoldKan/SplitSimplicialObject.lean,Mathlib/Analysis/InnerProductSpace/Laplacian.lean,Mathlib/Analysis/Normed/Field/Lemmas.lean,Mathlib/Analysis/Seminorm.lean,Mathlib/Analysis/SpecialFunctions/Gaussian/FourierTransform.lean,Mathlib/CategoryTheory/ComposableArrows.lean,Mathlib/CategoryTheory/Extensive.lean,Mathlib/CategoryTheory/FiberedCategory/Cocartesian.lean,Mathlib/CategoryTheory/Functor/Basic.lean,Mathlib/CategoryTheory/Functor/KanExtension/Preserves.lean,Mathlib/CategoryTheory/Functor/OfSequence.lean,Mathlib/CategoryTheory/Limits/Bicones.lean,Mathlib/CategoryTheory/Limits/Constructions/Over/Products.lean,Mathlib/CategoryTheory/Limits/Final/ParallelPair.lean,Mathlib/CategoryTheory/Limits/Preserves/Bifunctor.lean,Mathlib/CategoryTheory/Limits/Preserves/Shapes/Kernels.lean,Mathlib/CategoryTheory/Limits/Preserves/Shapes/Pullbacks.lean,Mathlib/CategoryTheory/Limits/Shapes/Equalizers.lean,Mathlib/CategoryTheory/Limits/Shapes/FiniteLimits.lean,Mathlib/CategoryTheory/Limits/Shapes/Multiequalizer.lean,Mathlib/CategoryTheory/Limits/Shapes/WideEqualizers.lean,Mathlib/CategoryTheory/Limits/Types/Shapes.lean,Mathlib/CategoryTheory/Localization/Construction.lean,Mathlib/CategoryTheory/Localization/Pi.lean,Mathlib/CategoryTheory/Monoidal/Cartesian/FunctorCategory.lean,Mathlib/CategoryTheory/Monoidal/DayConvolution.lean,Mathlib/CategoryTheory/Sites/MayerVietorisSquare.lean,Mathlib/Combinatorics/SimpleGraph/Regularity/Uniform.lean,Mathlib/Combinatorics/SimpleGraph/Triangle/Removal.lean,Mathlib/Computability/AkraBazzi/AkraBazzi.lean,Mathlib/Computability/AkraBazzi/GrowsPolynomially.lean,Mathlib/Computability/AkraBazzi/SumTransform.lean,Mathlib/Computability/TuringMachine.lean,Mathlib/Control/ULiftable.lean,Mathlib/Data/Bool/Basic.lean,Mathlib/Data/Fin/Fin2.lean,Mathlib/Data/Finmap.lean,Mathlib/Data/Finset/Card.lean,Mathlib/Data/Finset/Insert.lean,Mathlib/Data/Finset/Lattice/Basic.lean,Mathlib/Data/Finsupp/Option.lean,Mathlib/Data/Fintype/Fin.lean,Mathlib/Data/Int/Bitwise.lean,Mathlib/Data/Int/Cast/Defs.lean,Mathlib/Data/List/Basic.lean,Mathlib/Data/List/Chain.lean,Mathlib/Data/List/Destutter.lean,Mathlib/Data/List/Indexes.lean,Mathlib/Data/List/Nodup.lean,Mathlib/Data/List/Perm/Basic.lean,Mathlib/Data/List/Rotate.lean,Mathlib/Data/List/TakeWhile.lean,Mathlib/Data/Matrix/Notation.lean,Mathlib/Data/Multiset/Basic.lean,Mathlib/Data/Multiset/UnionInter.lean,Mathlib/Data/Nat/Bits.lean,Mathlib/Data/Nat/Cast/Defs.lean,Mathlib/Data/Nat/Cast/Order/Ring.lean,Mathlib/Data/Nat/Choose/Basic.lean,Mathlib/Data/Nat/Factorial/SuperFactorial.lean,Mathlib/Data/Nat/Fib/Basic.lean,Mathlib/Data/Nat/Find.lean,Mathlib/Data/Nat/Init.lean |
266 |
18 |
['MichaelStollBayreuth', 'adomani', 'github-actions', 'grunweg', 'leanprover-community-bot-assistant'] |
nobody |
43-81435 1 month ago |
43-81435 1 month ago |
0-0 0 seconds |
9935 |
jstoobysmith author:jstoobysmith |
feat(AlgebraicTopology): add constructors for horns |
Added a function that given a simplicial set S and a set of n-1 simplexes satisfying certain conditions, creates a morphism in SSet from a n horn to a simplicial set S.
Included also are a series of lemmas and definitions used in this construction. In particular I define a function that takes a m-simplex in a horn, and returns the smallest 'index' of face it factors through, and give a series of lemmas related to this.
---
[](https://gitpod.io/from-referrer/)
|
t-algebraic-topology
new-contributor
merge-conflict
awaiting-author
|
462/2 |
Mathlib/AlgebraicTopology/SimplicialSet.lean |
1 |
15 |
['YaelDillies', 'jcommelin', 'jstoobysmith', 'kim-em', 'linesthatinterlace'] |
nobody |
43-81165 1 month ago |
43-81165 1 month ago |
14-58814 14 days |
25914 |
eric-wieser author:eric-wieser |
feat: add an ext lemma for the opposite category |
This powers up `aesop_cat`.
---
[](https://gitpod.io/from-referrer/)
|
t-category-theory
awaiting-CI
merge-conflict
awaiting-author
|
18/56 |
Mathlib/AlgebraicTopology/SimplicialObject/Basic.lean,Mathlib/CategoryTheory/Abelian/Opposite.lean,Mathlib/CategoryTheory/Category/RelCat.lean,Mathlib/CategoryTheory/GuitartExact/Opposite.lean,Mathlib/CategoryTheory/Limits/Opposites.lean,Mathlib/CategoryTheory/Limits/Shapes/Products.lean,Mathlib/CategoryTheory/Opposites.lean,Mathlib/CategoryTheory/Triangulated/Opposite/Functor.lean,Mathlib/Combinatorics/Quiver/Basic.lean |
9 |
7 |
['eric-wieser', 'github-actions', 'grunweg', 'leanprover-community-bot-assistant', 'robin-carlier'] |
nobody |
43-79407 1 month ago |
70-22927 2 months ago |
1-77289 1 day |
20208 |
js2357 author:js2357 |
feat: Define the localization of a fractional ideal at a prime ideal |
Define the localization of a fractional ideal at a prime ideal, and prove some basic properties.
---
Alternate version of #14237 generalized to use `IsLocalization` and `IsFractionRing` rather than `Localization.AtPrime` and `FractionRing`
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
WIP
label:t-algebra$ |
248/0 |
Mathlib.lean,Mathlib/RingTheory/FractionalIdeal/LocalizedAtPrime.lean |
2 |
2 |
['github-actions', 'leanprover-community-bot-assistant'] |
nobody |
43-64650 1 month ago |
43-64651 1 month ago |
0-21 21 seconds |
19415 |
vihdzp author:vihdzp |
chore: move results on `Σ i : Fin n, f i` earlier |
---
[](https://gitpod.io/from-referrer/)
|
t-data
awaiting-CI
merge-conflict
|
131/145 |
Mathlib/Algebra/BigOperators/Fin.lean,Mathlib/Algebra/BigOperators/Finsupp.lean,Mathlib/Algebra/MvPolynomial/Equiv.lean,Mathlib/Algebra/Order/Antidiag/Pi.lean,Mathlib/Algebra/Polynomial/EraseLead.lean,Mathlib/AlgebraicTopology/AlternatingFaceMapComplex.lean,Mathlib/Combinatorics/Enumerative/Catalan.lean,Mathlib/Combinatorics/Optimization/ValuedCSP.lean,Mathlib/Data/Fin/Tuple/NatAntidiagonal.lean,Mathlib/Data/Fin/Tuple/Reflection.lean,Mathlib/Data/Fintype/BigOperators.lean,Mathlib/Data/Nat/Choose/Multinomial.lean,Mathlib/LinearAlgebra/LinearIndependent.lean |
13 |
4 |
['YaelDillies', 'github-actions', 'grunweg', 'vihdzp'] |
nobody |
43-54952 1 month ago |
285-6690 9 months ago |
0-0 0 seconds |
24260 |
plp127 author:plp127 |
feat(Topology): add API for Hereditarily Lindelof spaces |
Copies the stuff about Lindelof spaces to Hereditarily Lindelof spaces.
---
[](https://gitpod.io/from-referrer/)
|
t-topology
merge-conflict
awaiting-author
|
222/42 |
Mathlib/Topology/Compactness/Lindelof.lean |
1 |
15 |
['github-actions', 'grunweg', 'mathlib4-merge-conflict-bot', 'urkud'] |
urkud assignee:urkud |
43-34222 1 month ago |
43-34223 1 month ago |
29-42365 29 days |
27181 |
ADedecker author:ADedecker |
chore: more conceptual definition of `ValuativeRel.ValueGroupWithZero` |
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebra
merge-conflict
label:t-algebra$ |
685/467 |
Mathlib.lean,Mathlib/Data/Quot.lean,Mathlib/Data/Setoid/Basic.lean,Mathlib/GroupTheory/Congruence/Defs.lean,Mathlib/GroupTheory/Congruence/GroupWithZero.lean,Mathlib/RingTheory/OreLocalization/Basic.lean,Mathlib/RingTheory/OreLocalization/NonZeroDivisors.lean,Mathlib/RingTheory/OreLocalization/Ring.lean,Mathlib/RingTheory/Valuation/ValuativeRel.lean |
9 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-merge-conflict-bot'] |
nobody |
43-34211 1 month ago |
43-34212 1 month ago |
0-0 0 seconds |
27608 |
RemyDegenne author:RemyDegenne |
feat(MeasureTheory): typeclasses for measures with finite moments |
WIP because it seems useful for #26291 but I want to investigate more.
---
[](https://gitpod.io/from-referrer/)
|
t-measure-probability
merge-conflict
WIP
|
97/17 |
Mathlib.lean,Mathlib/MeasureTheory/Measure/Typeclasses/FiniteMoments.lean,Mathlib/Probability/Moments/CovarianceBilin.lean |
3 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
42-69087 1 month ago |
42-69088 1 month ago |
0-1 1 second |
26306 |
j-loreaux author:j-loreaux |
refactor: make `IsSelfAdjoint` and `IsIdempotentElem` one-field structures. |
---
[](https://gitpod.io/from-referrer/)
|
large-import
merge-conflict
|
222/224 |
Mathlib/Algebra/Algebra/Subalgebra/Pointwise.lean,Mathlib/Algebra/Algebra/Unitization.lean,Mathlib/Algebra/DirectSum/Idempotents.lean,Mathlib/Algebra/Group/Idempotent.lean,Mathlib/Algebra/Group/Submonoid/Membership.lean,Mathlib/Algebra/GroupWithZero/Idempotent.lean,Mathlib/Algebra/Order/Ring/Idempotent.lean,Mathlib/Algebra/Order/Ring/Star.lean,Mathlib/Algebra/Order/Star/Basic.lean,Mathlib/Algebra/Ring/BooleanRing.lean,Mathlib/Algebra/Ring/Idempotent.lean,Mathlib/Algebra/Star/Module.lean,Mathlib/Algebra/Star/SelfAdjoint.lean,Mathlib/Algebra/Star/StarProjection.lean,Mathlib/AlgebraicGeometry/Limits.lean,Mathlib/AlgebraicGeometry/Morphisms/FormallyUnramified.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Basic.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Order.lean,Mathlib/Analysis/CStarAlgebra/Module/Defs.lean,Mathlib/Analysis/InnerProductSpace/Adjoint.lean,Mathlib/Analysis/InnerProductSpace/LinearPMap.lean,Mathlib/Analysis/InnerProductSpace/Positive.lean,Mathlib/Analysis/InnerProductSpace/Projection.lean,Mathlib/Analysis/Normed/Algebra/Exponential.lean,Mathlib/Analysis/NormedSpace/MStructure.lean,Mathlib/Analysis/RCLike/Basic.lean,Mathlib/Data/Complex/Module.lean,Mathlib/LinearAlgebra/Matrix/Hermitian.lean,Mathlib/LinearAlgebra/Matrix/HermitianFunctionalCalculus.lean,Mathlib/LinearAlgebra/Matrix/PosDef.lean,Mathlib/LinearAlgebra/Projection.lean,Mathlib/LinearAlgebra/Span/Basic.lean,Mathlib/NumberTheory/NumberField/Completion.lean,Mathlib/NumberTheory/NumberField/InfinitePlace/Basic.lean,Mathlib/NumberTheory/NumberField/InfinitePlace/Embeddings.lean,Mathlib/NumberTheory/NumberField/InfinitePlace/Ramification.lean,Mathlib/RingTheory/DedekindDomain/Ideal.lean,Mathlib/RingTheory/Filtration.lean,Mathlib/RingTheory/Ideal/Cotangent.lean,Mathlib/RingTheory/Ideal/IdempotentFG.lean,Mathlib/RingTheory/Ideal/Span.lean,Mathlib/RingTheory/Idempotents.lean,Mathlib/RingTheory/Localization/Away/Basic.lean,Mathlib/RingTheory/Spectrum/Prime/Topology.lean,Mathlib/RingTheory/Unramified/Field.lean,Mathlib/RingTheory/Unramified/Finite.lean,Mathlib/RingTheory/Unramified/Pi.lean,Mathlib/Topology/Algebra/Module/LinearMap.lean |
48 |
6 |
['github-actions', 'j-loreaux', 'leanprover-community-bot-assistant', 'themathqueen'] |
nobody |
42-68853 1 month ago |
44-14932 1 month ago |
37-45446 37 days |
25726 |
tb65536 author:tb65536 |
(WIP) Galois group of `x ^ n - x - 1` |
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebra
merge-conflict
WIP
label:t-algebra$ |
512/145 |
Archive/Wiedijk100Theorems/AbelRuffini.lean,Mathlib/RingTheory/Polynomial/Selmer.lean |
2 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-merge-conflict-bot'] |
nobody |
41-3777 1 month ago |
41-3777 1 month ago |
0-1 1 second |
26344 |
mans0954 author:mans0954 |
feature(Analysis/NormedSpace/MStructure): The component projections on WithLp 1 (α × β) are L-projections |
This PR continues the work from #20380.
Original PR: https://github.com/leanprover-community/mathlib4/pull/20380 |
file-removed
t-analysis
merge-conflict
WIP
|
20/1 |
Mathlib.lean,Mathlib/Analysis/Normed/Lp/MStructure.lean,Mathlib/Analysis/Normed/Lp/ProdLp.lean |
3 |
3 |
['github-actions', 'mans0954', 'mathlib4-merge-conflict-bot'] |
nobody |
41-3529 1 month ago |
41-3530 1 month ago |
5-43696 5 days |
27870 |
grunweg author:grunweg |
draft: commandStart more --- fixing grounds |
A version of #26926 where I can slowly work towards fixing some violations.
---
[](https://gitpod.io/from-referrer/)
|
large-import
merge-conflict
WIP
|
2981/906 |
Mathlib/Algebra/Category/ModuleCat/ChangeOfRings.lean,Mathlib/Algebra/Divisibility/Basic.lean,Mathlib/Algebra/EuclideanDomain/Basic.lean,Mathlib/Algebra/Group/Commute/Defs.lean,Mathlib/Algebra/Group/Hom/CompTypeclasses.lean,Mathlib/Algebra/Group/Pointwise/Finset/Basic.lean,Mathlib/Algebra/Group/Semiconj/Basic.lean,Mathlib/Algebra/Group/Semiconj/Units.lean,Mathlib/Algebra/Homology/HomotopyCategory/HomComplex.lean,Mathlib/Algebra/Homology/HomotopyCategory/HomComplexShift.lean,Mathlib/Algebra/MvPolynomial/Equiv.lean,Mathlib/Algebra/Notation/Defs.lean,Mathlib/Algebra/Notation/Pi.lean,Mathlib/Algebra/Order/Antidiag/Pi.lean,Mathlib/Algebra/Polynomial/Laurent.lean,Mathlib/Algebra/Polynomial/Sequence.lean,Mathlib/Algebra/Polynomial/Smeval.lean,Mathlib/Algebra/Quaternion.lean,Mathlib/Algebra/Ring/Ext.lean,Mathlib/Analysis/InnerProductSpace/Laplacian.lean,Mathlib/Analysis/Seminorm.lean,Mathlib/Analysis/SpecialFunctions/Gaussian/FourierTransform.lean,Mathlib/CategoryTheory/FiberedCategory/Cocartesian.lean,Mathlib/CategoryTheory/Functor/Basic.lean,Mathlib/CategoryTheory/Functor/KanExtension/Preserves.lean,Mathlib/CategoryTheory/Limits/Preserves/Bifunctor.lean,Mathlib/CategoryTheory/Limits/Types/Shapes.lean,Mathlib/CategoryTheory/Monoidal/DayConvolution.lean,Mathlib/Combinatorics/SimpleGraph/Regularity/Uniform.lean,Mathlib/Combinatorics/SimpleGraph/Triangle/Removal.lean,Mathlib/Computability/AkraBazzi/AkraBazzi.lean,Mathlib/Computability/AkraBazzi/GrowsPolynomially.lean,Mathlib/Computability/AkraBazzi/SumTransform.lean,Mathlib/Computability/TuringMachine.lean,Mathlib/Control/ULiftable.lean,Mathlib/Data/Bool/Basic.lean,Mathlib/Data/Fin/Fin2.lean,Mathlib/Data/Finmap.lean,Mathlib/Data/Finset/Card.lean,Mathlib/Data/Finset/Lattice/Basic.lean,Mathlib/Data/Fintype/Fin.lean,Mathlib/Data/Int/Bitwise.lean,Mathlib/Data/Int/Cast/Defs.lean,Mathlib/Data/List/Basic.lean,Mathlib/Data/List/Chain.lean,Mathlib/Data/List/Destutter.lean,Mathlib/Data/List/Indexes.lean,Mathlib/Data/List/Nodup.lean,Mathlib/Data/List/Perm/Basic.lean,Mathlib/Data/List/Rotate.lean,Mathlib/Data/List/TakeWhile.lean,Mathlib/Data/Matrix/Notation.lean,Mathlib/Data/Multiset/Basic.lean,Mathlib/Data/Multiset/UnionInter.lean,Mathlib/Data/Nat/Bits.lean,Mathlib/Data/Nat/Cast/Defs.lean,Mathlib/Data/Nat/Choose/Basic.lean,Mathlib/Data/Nat/Factorial/SuperFactorial.lean,Mathlib/Data/Nat/Log.lean,Mathlib/Data/Option/Basic.lean,Mathlib/Data/PSigma/Order.lean,Mathlib/Data/Part.lean,Mathlib/Data/Prod/Basic.lean,Mathlib/Data/Real/Pi/Bounds.lean,Mathlib/Data/Seq/Computation.lean,Mathlib/Data/Seq/Seq.lean,Mathlib/Data/Set/Basic.lean,Mathlib/Data/Set/Defs.lean,Mathlib/Data/Set/Function.lean,Mathlib/Data/Sigma/Order.lean,Mathlib/Data/Stream/Init.lean,Mathlib/Data/Sum/Basic.lean,Mathlib/Data/Sym/Sym2.lean,Mathlib/Data/TypeVec.lean,Mathlib/Data/Vector/Basic.lean,Mathlib/Geometry/Manifold/PoincareConjecture.lean,Mathlib/Geometry/Manifold/VectorBundle/SmoothSection.lean,Mathlib/GroupTheory/ArchimedeanDensely.lean,Mathlib/GroupTheory/CoprodI.lean,Mathlib/GroupTheory/Coxeter/Basic.lean,Mathlib/GroupTheory/Coxeter/Inversion.lean,Mathlib/GroupTheory/Coxeter/Length.lean,Mathlib/GroupTheory/FixedPointFree.lean,Mathlib/GroupTheory/GroupAction/Blocks.lean,Mathlib/GroupTheory/GroupAction/MultipleTransitivity.lean,Mathlib/GroupTheory/GroupAction/Primitive.lean,Mathlib/GroupTheory/GroupAction/SubMulAction/OfFixingSubgroup.lean,Mathlib/GroupTheory/HNNExtension.lean,Mathlib/GroupTheory/MonoidLocalization/Basic.lean,Mathlib/GroupTheory/MonoidLocalization/MonoidWithZero.lean,Mathlib/GroupTheory/Perm/Centralizer.lean,Mathlib/GroupTheory/Perm/Cycle/Concrete.lean,Mathlib/GroupTheory/Perm/DomMulAct.lean,Mathlib/GroupTheory/PushoutI.lean,Mathlib/GroupTheory/SpecificGroups/Dihedral.lean,Mathlib/GroupTheory/SpecificGroups/Quaternion.lean,Mathlib/LinearAlgebra/BilinearForm/TensorProduct.lean,Mathlib/LinearAlgebra/CliffordAlgebra/EvenEquiv.lean,Mathlib/LinearAlgebra/CliffordAlgebra/Prod.lean,Mathlib/LinearAlgebra/Eigenspace/Matrix.lean |
202 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
40-86086 1 month ago |
40-86087 1 month ago |
0-0 0 seconds |
27445 |
erdOne author:erdOne |
chore(RingTheory/LocalRing): fix problematic instance |
We shouldn't use `RingHom.toAlgebra` for `Algebra (ResidueField R) (ResidueField S)`. The smul should come from the smul field in `Algebra`.
- Redefined `Algebra (ResidueField R) (ResidueField S)` via `Ideal.Quotient.algebraOfLiesOver`, and provided missing `IsScalarTower` instances for it.
- Added missing `IsScalarTower` for `Localization.AtPrime`.
- Removed `Algebra p.ResidueField q.ResidueField` and the `IsScalarTower` instances coming with it (because there are `inferInstance` now)
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
label:t-algebra$ |
37/37 |
Mathlib/Algebra/Order/Archimedean/Submonoid.lean,Mathlib/RingTheory/LocalRing/ResidueField/Algebraic.lean,Mathlib/RingTheory/LocalRing/ResidueField/Basic.lean,Mathlib/RingTheory/LocalRing/ResidueField/Ideal.lean,Mathlib/RingTheory/LocalRing/ResidueField/Instances.lean,Mathlib/RingTheory/Localization/AtPrime.lean,Mathlib/RingTheory/Unramified/LocalRing.lean |
7 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
40-54219 1 month ago |
40-54219 1 month ago |
9-82484 9 days |
27267 |
JovanGerb author:JovanGerb |
chore(Order): refactor in preparation for `to_dual` |
WIP
---
[](https://gitpod.io/from-referrer/)
|
t-order
merge-conflict
|
60/52 |
Mathlib/Data/Nat/Find.lean,Mathlib/Order/Basic.lean,Mathlib/Order/Defs/LinearOrder.lean,Mathlib/Order/Defs/PartialOrder.lean,Mathlib/Tactic/Linarith/Frontend.lean,Mathlib/Tactic/Positivity/Core.lean |
6 |
2 |
['github-actions', 'leanprover-community-bot-assistant'] |
bryangingechen assignee:bryangingechen |
40-2383 1 month ago |
40-2388 1 month ago |
0-0 0 seconds |
26383 |
eric-wieser author:eric-wieser |
feat: `Real.sin_eq_one_iff` and similar |
---
[](https://gitpod.io/from-referrer/)
|
t-analysis
merge-conflict
|
155/101 |
Mathlib/Algebra/ModEq.lean,Mathlib/Analysis/SpecialFunctions/Complex/Log.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Angle.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Basic.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Complex.lean |
5 |
2 |
['github-actions', 'leanprover-community-bot-assistant'] |
nobody |
40-1915 1 month ago |
40-1915 1 month ago |
0-0 0 seconds |
26010 |
linesthatinterlace author:linesthatinterlace |
feat(`Algebra/Group/Prod`): Add API for inclusion and projection maps from and to the product of units. |
This PR continues the work from #25112.
Original PR: https://github.com/leanprover-community/mathlib4/pull/25112 |
migrated-from-branch
t-algebra
merge-conflict
WIP
label:t-algebra$ |
292/122 |
Mathlib.lean,Mathlib/Algebra/BigOperators/Associated.lean,Mathlib/Algebra/BigOperators/Group/Finset/Defs.lean,Mathlib/Algebra/Group/Commute/Units.lean,Mathlib/Algebra/Group/Prod.lean,Mathlib/Algebra/Group/Semiconj/Units.lean,Mathlib/Algebra/Group/Subgroup/Ker.lean,Mathlib/Algebra/Group/Units/Defs.lean,Mathlib/Algebra/Group/Units/Hom.lean,Mathlib/Algebra/Group/Units/Prod.lean,Mathlib/Algebra/Star/SelfAdjoint.lean,Mathlib/Data/Nat/Totient.lean,Mathlib/Topology/Algebra/Group/Basic.lean |
13 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'linesthatinterlace'] |
nobody |
40-1806 1 month ago |
40-1806 1 month ago |
0-2113 35 minutes |
25991 |
Multramate author:Multramate |
feat(AlgebraicGeometry/EllipticCurve): generalise nonsingular condition |
This PR continues the work from #25219.
Original PR: https://github.com/leanprover-community/mathlib4/pull/25219 |
t-algebraic-geometry
merge-conflict
|
2127/1561 |
Mathlib/Algebra/Group/Units/Basic.lean,Mathlib/Algebra/Group/Units/Hom.lean,Mathlib/Algebra/Module/PID.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Affine/Basic.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Affine/Formula.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Affine/Point.lean,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,Mathlib/RingTheory/DedekindDomain/AdicValuation.lean,Mathlib/RingTheory/Ideal/Maps.lean,Mathlib/RingTheory/Ideal/Span.lean |
15 |
n/a |
['github-actions', 'leanprover-community-bot-assistant'] |
nobody |
40-1797 1 month ago |
unknown |
unknown |
25985 |
Multramate author:Multramate |
feat(AlgebraicGeometry/EllipticCurve/Jacobian): add equivalences between points and explicit WithZero types |
This PR continues the work from #14923.
Original PR: https://github.com/leanprover-community/mathlib4/pull/14923 |
t-algebraic-geometry
merge-conflict
|
262/66 |
Mathlib/AlgebraicGeometry/EllipticCurve/Affine.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Group.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Jacobian.lean,scripts/style-exceptions.txt |
4 |
1 |
['Multramate'] |
nobody |
40-1785 1 month ago |
40-1785 1 month ago |
0-48 48 seconds |
25984 |
Multramate author:Multramate |
feat(AlgebraicGeometry/EllipticCurve/Affine): add equivalences between points and explicit WithZero types |
This PR continues the work from #14627.
Original PR: https://github.com/leanprover-community/mathlib4/pull/14627 |
t-algebraic-geometry
merge-conflict
|
159/52 |
Mathlib/AlgebraicGeometry/EllipticCurve/Affine.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Group.lean |
2 |
1 |
['Multramate'] |
nobody |
40-1781 1 month ago |
40-1781 1 month ago |
0-55 55 seconds |
25983 |
Multramate author:Multramate |
feat(AlgebraicGeometry/EllipticCurve/Scheme): define the affine scheme associated to an elliptic curve |
This PR continues the work from #14130.
Original PR: https://github.com/leanprover-community/mathlib4/pull/14130 |
t-algebraic-geometry
merge-conflict
|
557/22 |
Mathlib/Algebra/DirectSum/Basic.lean,Mathlib/Algebra/DirectSum/Module.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Scheme.lean,Mathlib/RingTheory/GradedAlgebra/Basic.lean,Mathlib/RingTheory/MvPolynomial/Homogeneous.lean,Mathlib/RingTheory/MvPolynomial/WeightedHomogeneous.lean |
6 |
1 |
['Multramate'] |
nobody |
40-1776 1 month ago |
40-1776 1 month ago |
0-0 0 seconds |
25982 |
Multramate author:Multramate |
feat(AlgebraicGeometry/EllipticCurve/Group): compute range of baseChange |
This PR continues the work from #10142.
Original PR: https://github.com/leanprover-community/mathlib4/pull/10142 |
t-algebraic-geometry
merge-conflict
|
421/212 |
Mathlib/AlgebraicGeometry/EllipticCurve/Affine.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Group.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Weierstrass.lean,Mathlib/GroupTheory/GroupAction/Basic.lean,Mathlib/GroupTheory/Subgroup/Basic.lean,Mathlib/GroupTheory/Submonoid/Operations.lean |
6 |
1 |
['Multramate'] |
nobody |
40-1771 1 month ago |
40-1771 1 month ago |
0-57 57 seconds |
25981 |
Multramate author:Multramate |
feat(GroupTheory/GroupAction/Basic): define homomorphisms of fixed subgroups induced by homomorphisms of groups |
This PR continues the work from #10126.
Original PR: https://github.com/leanprover-community/mathlib4/pull/10126 |
t-group-theory
merge-conflict
|
81/12 |
Mathlib/GroupTheory/GroupAction/Basic.lean,Mathlib/GroupTheory/Subgroup/Basic.lean,Mathlib/GroupTheory/Submonoid/Operations.lean |
3 |
0 |
[] |
nobody |
40-1765 1 month ago |
40-1765 1 month ago |
0-52 52 seconds |
25980 |
Multramate author:Multramate |
feat(GroupTheory/Submonoid/Operations): define homomorphisms of subgroups induced by homomorphisms of groups |
This PR continues the work from #10113.
Original PR: https://github.com/leanprover-community/mathlib4/pull/10113 |
t-group-theory
merge-conflict
|
29/6 |
Mathlib/GroupTheory/Subgroup/Basic.lean,Mathlib/GroupTheory/Submonoid/Operations.lean |
2 |
0 |
[] |
nobody |
40-1760 1 month ago |
40-1760 1 month ago |
0-54 54 seconds |
25485 |
VTrelat author:VTrelat |
feat(SetTheory/ZFC/Naturals): define natural numbers in ZFC |
Extend the model of ZFC with naturals:
- define a set `Nat` of naturals following the usual construction (∅, {∅}, {∅, {∅}}, ...)
- define a proper type `ZFNat` representing naturals
- add theorems on usual algebraic properties of naturals
- provide a recursor and induction schemes to define/prove by induction
---
[](https://gitpod.io/from-referrer/)
- [ ] depend on: #25483
|
t-set-theory
new-contributor
merge-conflict
|
2095/0 |
Mathlib/Data/Set/Prod.lean,Mathlib/SetTheory/ZFC/Basic.lean,Mathlib/SetTheory/ZFC/Booleans.lean,Mathlib/SetTheory/ZFC/Naturals.lean |
4 |
2 |
['github-actions', 'leanprover-community-bot-assistant'] |
nobody |
40-1585 1 month ago |
40-1585 1 month ago |
29-51653 29 days |
25474 |
adomani author:adomani |
test for .lean/.md check |
A test PR for #25473.
---
[](https://gitpod.io/from-referrer/)
|
file-removed
t-linter
merge-conflict
|
10/1 |
.github/workflows/lint_and_suggest_pr.yml,Mathlib.lean,Mathlib/NumberTheory/NumberField/CMField.Lean |
3 |
2 |
['github-actions', 'leanprover-community-bot-assistant'] |
nobody |
40-1574 1 month ago |
40-1574 1 month ago |
29-67280 29 days |
25425 |
Paul-Lez author:Paul-Lez |
feat(LinearAlgebra/Basis/HasCanonicalBasis): propose `HasCanonicalBasis` class |
Context: in some cases, e.g. writing down PDEs, having a notion of partial derivatives can be useful. In an ideal world (as mentioned by @ocfnash in [this Zulip thread](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Partial.20derivatives/with/463936246)), one could write something along the lines of `open scoped PartialDerivatives` in order to access nice notation for this.
This PR introduces a notion of a canonical basis for a module in order to allow taking partial derivatives with respect to it.
A later PR (which I am about open) would then propose a notation for taking partial derivatives (defined using `lineDeriv` in order to avoid requiring Frechet-differentiability assumptions). The goal here is to have notation that works equally well on e.g. `𝕜 × 𝕜` and `EuclideanSpace 𝕜 (Fin 2)` and so on.
I've opened this PR as a draft in order to get some initial feedback on the content (and whether this is considered appropriate for Mathlib!); the file itself would need to be split (e.g. the instances defined should probably go in different files)
Co-authored-by: Eric Wieser
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
label:t-algebra$ |
105/0 |
Mathlib.lean,Mathlib/LinearAlgebra/Basis/HasCanonicalBasis.lean |
2 |
2 |
['github-actions', 'leanprover-community-bot-assistant'] |
nobody |
40-1565 1 month ago |
40-1565 1 month ago |
0-0 0 seconds |
25362 |
adomani author:adomani |
feat: a linter for duplicated `open` |
This linter warns when a namespace is repeated.
It makes an effort to report only the problematic namespaces, but is not especially robust. The linter has some awareness of the `namespace` command, so
```lean
def X.Y := 0
open X
namespace X
open Y
```
will flag both `namespace X` and `open Y` as problematic, even though it was the `open `X` that became redundant with `namespace X`.
However, I will not have much time to devote to polishing this and there are quite a few exception in Mathlib before a better version could be seriously considered for adoption.
[#mathlib4 > linter requests @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/linter.20requests/near/520273644)
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-linter
merge-conflict
please-adopt
|
191/94 |
Mathlib.lean,Mathlib/Algebra/Group/Pi/Basic.lean,Mathlib/Algebra/GroupWithZero/Pi.lean,Mathlib/Algebra/Order/Ring/InjSurj.lean,Mathlib/CategoryTheory/Functor/ReflectsIso/Basic.lean,Mathlib/Data/Fin/Basic.lean,Mathlib/Data/Finite/Defs.lean,Mathlib/Data/Ineq.lean,Mathlib/Data/List/Lemmas.lean,Mathlib/Data/List/NatAntidiagonal.lean,Mathlib/Data/Nat/Choose/Basic.lean,Mathlib/Data/Nat/Prime/Basic.lean,Mathlib/Data/Nat/Prime/Defs.lean,Mathlib/Data/Set/Image.lean,Mathlib/Data/Set/Insert.lean,Mathlib/Init.lean,Mathlib/Logic/Basic.lean,Mathlib/Logic/Embedding/Set.lean,Mathlib/Logic/Pairwise.lean,Mathlib/Order/BoundedOrder/Basic.lean,Mathlib/Order/WithBot.lean,Mathlib/RingTheory/OreLocalization/Basic.lean,Mathlib/Tactic.lean,Mathlib/Tactic/ApplyFun.lean,Mathlib/Tactic/Bound.lean,Mathlib/Tactic/CongrM.lean,Mathlib/Tactic/Find.lean,Mathlib/Tactic/Lift.lean,Mathlib/Tactic/Linarith/Oracle/FourierMotzkin.lean,Mathlib/Tactic/Linter.lean,Mathlib/Tactic/Linter/DupOpen.lean,Mathlib/Tactic/NormNum/PowMod.lean,Mathlib/Tactic/Recover.lean,Mathlib/Tactic/ReduceModChar.lean,Mathlib/Tactic/Widget/Calc.lean,Mathlib/Tactic/Widget/SelectInsertParamsClass.lean,Mathlib/Tactic/Widget/StringDiagram.lean,Mathlib/Topology/CWComplex/Abstract/Basic.lean,Mathlib/Topology/ContinuousMap/Interval.lean,Mathlib/Topology/Germ.lean,Mathlib/Topology/Homotopy/HSpaces.lean,Mathlib/Topology/Order/LowerUpperTopology.lean,Mathlib/Topology/Order/PartialSups.lean,Mathlib/Topology/Separation/DisjointCover.lean,Mathlib/Topology/Sheaves/Sheafify.lean,Mathlib/Util/CountHeartbeats.lean,MathlibTest/DupOpen.lean |
47 |
14 |
['adomani', 'github-actions', 'grunweg', 'leanprover-community-bot-assistant', 'mathlib4-merge-conflict-bot'] |
nobody |
40-1560 1 month ago |
40-1560 1 month ago |
0-0 0 seconds |
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
t-meta
merge-conflict
|
17/5 |
Mathlib/Tactic/ComputeDegree.lean,MathlibTest/ComputeDegree.lean |
2 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
40-1555 1 month ago |
40-1555 1 month ago |
38-26044 38 days |
17145 |
Command-Master author:Command-Master |
feat(Archive/Ioi/Ioi2024Q2): a proof of the solution of question 2 from IOI 2024. |
---
- [x] depends on: #17189
- [x] depends on: #17190
- [x] depends on: #17191
[](https://gitpod.io/from-referrer/)
|
large-import
IMO
merge-conflict
WIP
|
1013/1 |
Archive.lean,Archive/Ioi/Ioi2024Q2.lean,Mathlib.lean,Mathlib/Combinatorics/Orbits.lean,Mathlib/Data/List/SplitLengths.lean,Mathlib/Data/List/Transpose.lean,Mathlib/Data/List/Zip.lean,Mathlib/Data/Vector/Basic.lean,Mathlib/Data/Vector/Defs.lean,Mathlib/Data/Vector/MapLemmas.lean,Mathlib/Data/Vector/Transpose.lean,Mathlib/GroupTheory/Perm/Cycle/Basic.lean,Mathlib/Logic/Function/Iterate.lean,Mathlib/Order/Antisymmetrization.lean,Mathlib/Order/Partition/Finpartition.lean |
15 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
40-1515 1 month ago |
40-1515 1 month ago |
0-0 0 seconds |
14137 |
mattrobball author:mattrobball |
chore(Algebra.Basic): postpone importing algebra instances for `Nat`, `Int`, and `Rat` |
This should help typeclass synthesis by avoiding these instances unless absolutely necessary.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
label:t-algebra$ |
678/356 |
Counterexamples/Pseudoelement.lean,Mathlib.lean,Mathlib/Algebra/Algebra/Basic.lean,Mathlib/Algebra/Algebra/Bilinear.lean,Mathlib/Algebra/Algebra/Equiv.lean,Mathlib/Algebra/Algebra/Hom/Basic.lean,Mathlib/Algebra/Algebra/Hom/Int.lean,Mathlib/Algebra/Algebra/Hom/Nat.lean,Mathlib/Algebra/Algebra/Hom/Rat.lean,Mathlib/Algebra/Algebra/Int.lean,Mathlib/Algebra/Algebra/Nat.lean,Mathlib/Algebra/Algebra/NonUnitalHom.lean,Mathlib/Algebra/Algebra/NonUnitalSubalgebra.lean,Mathlib/Algebra/Algebra/Prod.lean,Mathlib/Algebra/Algebra/Rat.lean,Mathlib/Algebra/Algebra/Subalgebra/Basic.lean,Mathlib/Algebra/Algebra/Subalgebra/Int.lean,Mathlib/Algebra/Algebra/Subalgebra/Nat.lean,Mathlib/Algebra/Algebra/Subalgebra/Unitization.lean,Mathlib/Algebra/Algebra/Tower.lean,Mathlib/Algebra/FreeAlgebra.lean,Mathlib/Algebra/Group/AddChar.lean,Mathlib/Algebra/Module/Bimodule.lean,Mathlib/Algebra/Module/Zlattice/Basic.lean,Mathlib/Algebra/MonoidAlgebra/Basic.lean,Mathlib/Algebra/MvPolynomial/Counit.lean,Mathlib/Algebra/MvPolynomial/NatInt.lean,Mathlib/Algebra/MvPolynomial/Supported.lean,Mathlib/Algebra/Polynomial/AlgebraMap.lean,Mathlib/Algebra/Polynomial/DenomsClearable.lean,Mathlib/Algebra/Polynomial/Int.lean,Mathlib/Algebra/RingQuot.lean,Mathlib/Analysis/NormedSpace/Basic.lean,Mathlib/CategoryTheory/Galois/Examples.lean,Mathlib/Data/Complex/Module.lean,Mathlib/Data/Real/Irrational.lean,Mathlib/FieldTheory/IsAlgClosed/AlgebraicClosure.lean,Mathlib/FieldTheory/SplittingField/Construction.lean,Mathlib/LinearAlgebra/Matrix/Adjugate.lean,Mathlib/LinearAlgebra/Prod.lean,Mathlib/NumberTheory/ClassNumber/AdmissibleAbs.lean,Mathlib/NumberTheory/NumberField/Basic.lean,Mathlib/NumberTheory/NumberField/Embeddings.lean,Mathlib/RingTheory/Adjoin/Basic.lean,Mathlib/RingTheory/Adjoin/FG.lean,Mathlib/RingTheory/Adjoin/NatInt.lean,Mathlib/RingTheory/AlgebraTower.lean,Mathlib/RingTheory/Bialgebra/Hom.lean,Mathlib/RingTheory/Coalgebra/Hom.lean,Mathlib/RingTheory/IntegralClosure.lean,Mathlib/RingTheory/Localization/Basic.lean,Mathlib/RingTheory/Localization/FractionRing.lean,Mathlib/RingTheory/Localization/FractionRingInt.lean,Mathlib/RingTheory/Localization/Int.lean,Mathlib/RingTheory/Localization/Nat.lean,Mathlib/RingTheory/Polynomial/GaussLemma.lean,Mathlib/RingTheory/Polynomial/Pochhammer.lean,Mathlib/RingTheory/PowerSeries/WellKnown.lean,Mathlib/RingTheory/TensorProduct/Basic.lean,Mathlib/RingTheory/WittVector/MulCoeff.lean,Mathlib/Topology/Algebra/Algebra.lean,Mathlib/Topology/Instances/Real.lean,test/infer_instance.lean,test/instance_diamonds.lean |
64 |
7 |
['fpvandoorn', 'github-actions', 'grunweg', 'leanprover-bot', 'mattrobball'] |
nobody |
40-1511 1 month ago |
40-1511 1 month ago |
0-0 0 seconds |
11632 |
mattrobball author:mattrobball |
chore(Group/RingTheory.Congruence): make `Quotient`'s reducible |
These are essentially wrappers and should not expose any data when made reducible. Their use in constructing typeclass instances makes reducible transparency desirable.
---
[](https://gitpod.io/from-referrer/)
|
t-group-theory
merge-conflict
|
16/35 |
Mathlib/GroupTheory/Congruence/Basic.lean,Mathlib/RingTheory/Congruence/Basic.lean |
2 |
14 |
['eric-wieser', 'fpvandoorn', 'github-actions', 'grunweg', 'kmill', 'leanprover-bot', 'mattrobball'] |
nobody |
40-1502 1 month ago |
40-1502 1 month ago |
2-10495 2 days |
3171 |
eric-wieser author:eric-wieser |
refactor: make the algebra hierarchy use flat structures |
By introducing a `FlatHack` base class and using it as the first parent of every algebra typeclass, it causes the typeclasses to all overlap and so we emulate flat structures.
Most of the pain here comes from `to_additive` not generating any of the ancestor projections properly; this was already a bug present for `n + 1` parents, but now the `1` is taken up
This is one workaround for leanprover/lean4#2074: don't let the eta-diamonds appear in the first place.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
WIP
label:t-algebra$ |
328/240 |
.github/workflows/build.yml,Mathlib/Algebra/Algebra/Equiv.lean,Mathlib/Algebra/Algebra/Hom.lean,Mathlib/Algebra/Category/GroupCat/Basic.lean,Mathlib/Algebra/Category/GroupCat/EquivalenceGroupAddGroup.lean,Mathlib/Algebra/Category/MonCat/FilteredColimits.lean,Mathlib/Algebra/DualNumber.lean,Mathlib/Algebra/Field/Defs.lean,Mathlib/Algebra/GCDMonoid/Basic.lean,Mathlib/Algebra/Group/Basic.lean,Mathlib/Algebra/Group/Defs.lean,Mathlib/Algebra/Group/Ext.lean,Mathlib/Algebra/Group/Opposite.lean,Mathlib/Algebra/Group/Prod.lean,Mathlib/Algebra/GroupPower/Lemmas.lean,Mathlib/Algebra/Hom/Group.lean,Mathlib/Algebra/MonoidAlgebra/Basic.lean,Mathlib/Algebra/Order/Chebyshev.lean,Mathlib/Algebra/Order/Group/Abs.lean,Mathlib/Algebra/Order/Group/Defs.lean,Mathlib/Algebra/Order/Module.lean,Mathlib/Algebra/Order/Rearrangement.lean,Mathlib/Algebra/Order/Ring/Canonical.lean,Mathlib/Algebra/Order/Ring/Defs.lean,Mathlib/Algebra/Quandle.lean,Mathlib/Algebra/Ring/Defs.lean,Mathlib/Algebra/TrivSqZeroExt.lean,Mathlib/CategoryTheory/Endomorphism.lean,Mathlib/CategoryTheory/Preadditive/Basic.lean,Mathlib/CategoryTheory/Preadditive/SingleObj.lean,Mathlib/Data/Finsupp/Multiset.lean,Mathlib/Data/Int/LeastGreatest.lean,Mathlib/Data/Int/Order/Basic.lean,Mathlib/Data/Int/Order/Lemmas.lean,Mathlib/Data/Nat/Choose/Multinomial.lean,Mathlib/Data/Real/CauSeqCompletion.lean,Mathlib/Data/ZMod/Defs.lean,Mathlib/LinearAlgebra/AffineSpace/Ordered.lean,Mathlib/LinearAlgebra/LinearPMap.lean,Mathlib/RingTheory/Ideal/Quotient.lean,Mathlib/Tactic/Positivity/Core.lean,Mathlib/Tactic/Ring/Basic.lean |
42 |
14 |
['eric-wieser', 'gebner', 'harahu'] |
nobody |
40-1497 1 month ago |
40-1497 1 month ago |
0-0 0 seconds |
26760 |
linesthatinterlace author:linesthatinterlace |
refactor(`InformationTheory/Hamming`): Improvements to Hamming type. |
Turns Hamming type into a structure with one field.
Per discussions in https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/defeq.20abuse.20in.20.60WithLp.60/with/462136240.
---
To remove the chance of defeq-abuse for the Hamming type, this refactors it as a structure with one field, and makes some other improvements while there.
[](https://gitpod.io/from-referrer/)
|
file-removed
t-measure-probability
merge-conflict
WIP
|
306/412 |
Mathlib/InformationTheory/Hamming.lean,Mathlib/InformationTheory/Hamming/Defs.lean,Mathlib/InformationTheory/Hamming/Group.lean,Mathlib/InformationTheory/Hamming/Module.lean,Mathlib/InformationTheory/Hamming/Norm.lean |
5 |
7 |
['eric-wieser', 'github-actions', 'linesthatinterlace', 'mathlib4-merge-conflict-bot'] |
nobody |
39-85900 1 month ago |
39-85901 1 month ago |
0-20107 5 hours |
27643 |
ADedecker author:ADedecker |
Ad bdd unif conv |
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict |
111/26 |
Mathlib/Analysis/LocallyConvex/Bounded.lean,Mathlib/Topology/Algebra/Module/StrongTopology.lean,Mathlib/Topology/Algebra/Module/UniformConvergence.lean,Mathlib/Topology/Bornology/Absorbs.lean |
4 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
39-66674 1 month ago |
39-66674 1 month ago |
0-0 0 seconds |
26385 |
jjdishere author:jjdishere |
feat(RingTheory/Perfectoid): define integral perfectoid rings |
This PR continues the work from #22331.
Original PR: https://github.com/leanprover-community/mathlib4/pull/22331 |
t-ring-theory
merge-conflict
WIP
|
1081/15 |
Mathlib.lean,Mathlib/Algebra/Ring/Aut.lean,Mathlib/FieldTheory/Perfect.lean,Mathlib/RingTheory/AdicCompletion/Basic.lean,Mathlib/RingTheory/Ideal/Maps.lean,Mathlib/RingTheory/Ideal/Quotient/Defs.lean,Mathlib/RingTheory/Ideal/Quotient/PowTransition.lean,Mathlib/RingTheory/Perfection.lean,Mathlib/RingTheory/Perfectoid/BDeRham.lean,Mathlib/RingTheory/Perfectoid/FontaineTheta.lean,Mathlib/RingTheory/Perfectoid/IntergalPerfectoid.lean,Mathlib/RingTheory/Perfectoid/Untilt.lean,Mathlib/RingTheory/WittVector/Basic.lean,Mathlib/RingTheory/WittVector/Complete.lean,Mathlib/RingTheory/WittVector/TeichmullerSeries.lean,docs/references.bib |
16 |
3 |
['github-actions', 'jjdishere', 'leanprover-community-bot-assistant'] |
nobody |
39-3982 1 month ago |
39-3983 1 month ago |
0-79 1 minute |
22898 |
AntoineChambert-Loir author:AntoineChambert-Loir |
feat(RingTheory/TensorProduct/DirectLimit/FG): direct limit of finitely generated submodules and tensor product |
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
merge-conflict
WIP
|
399/0 |
Mathlib.lean,Mathlib/RingTheory/Adjoin/FG.lean,Mathlib/RingTheory/Finiteness/Basic.lean,Mathlib/RingTheory/TensorProduct/Basic.lean,Mathlib/RingTheory/TensorProduct/DirectLimit/FG.lean |
5 |
9 |
['AntoineChambert-Loir', 'alreadydone', 'github-actions', 'leanprover-community-bot-assistant'] |
nobody |
39-3642 1 month ago |
39-3642 1 month ago |
11-9349 11 days |
21255 |
chrisflav author:chrisflav |
feat(RingTheory/Smooth): smooth is equivalent to locally standard smooth |
This is only a container to not lose the branch name.
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
merge-conflict
|
1740/11 |
Mathlib.lean,Mathlib/RingTheory/Kaehler/Localization.lean,Mathlib/RingTheory/Presentation.lean,Mathlib/RingTheory/Smooth/FreeKaehler.lean,Mathlib/RingTheory/Smooth/StandardSmoothCotangent.lean,Mathlib/RingTheory/Smooth/StandardSmoothSmooth.lean |
6 |
2 |
['github-actions', 'leanprover-community-bot-assistant'] |
nobody |
39-3605 1 month ago |
39-3605 1 month ago |
0-0 0 seconds |
20431 |
erdOne author:erdOne |
feat(RingTheory/AdicCompletion): monotonicity of adic-completeness |
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
merge-conflict
awaiting-author
|
206/16 |
Mathlib.lean,Mathlib/Algebra/Module/Submodule/Defs.lean,Mathlib/Algebra/Module/Submodule/Pointwise.lean,Mathlib/RingTheory/AdicCompletion/Algebra.lean,Mathlib/RingTheory/AdicCompletion/Basic.lean,Mathlib/RingTheory/AdicCompletion/Mono.lean,Mathlib/RingTheory/Finiteness/Ideal.lean |
7 |
13 |
['chrisflav', 'erdOne', 'github-actions'] |
nobody |
39-3598 1 month ago |
39-3598 1 month ago |
35-86379 35 days |
20424 |
erdOne author:erdOne |
feat(RingTheory): evaluation of power series |
---
- [ ] depends on: #20425
- [x] depends on: #20426
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
merge-conflict
|
425/8 |
Mathlib.lean,Mathlib/RingTheory/AdicCompletion/Noetherian.lean,Mathlib/RingTheory/Filtration.lean,Mathlib/RingTheory/PowerSeries/Basic.lean,Mathlib/RingTheory/PowerSeries/Eval.lean,Mathlib/RingTheory/PowerSeries/Trunc.lean |
6 |
11 |
['AntoineChambert-Loir', 'alreadydone', 'erdOne', 'eric-wieser', 'github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
39-3591 1 month ago |
39-3591 1 month ago |
0-3944 1 hour |
19596 |
Command-Master author:Command-Master |
feat(RingTheory/Valuation/PrimeMultiplicity): define `WithTop ℤ`-valued prime multiplicity on a fraction field |
Moves:
- `multiplicity_addValuation` -> `AddValuation.multiplicity`
- `multiplicity_addValuation_apply` -> `AddValuation.multiplicity_apply`
---
- [x] depends on: #19149
- [x] depends on: #18786
- [x] depends on: #19122
- [x] depends on: #18954
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
large-import
merge-conflict
awaiting-author
|
101/37 |
Mathlib/Data/ENat/Basic.lean,Mathlib/RingTheory/DiscreteValuationRing/Basic.lean,Mathlib/RingTheory/Valuation/PrimeMultiplicity.lean |
3 |
11 |
['ChrisHughes24', 'Command-Master', 'Vierkantor', 'faenuccio', 'github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
39-3583 1 month ago |
39-3583 1 month ago |
8-2214 8 days |
18646 |
jxjwan author:jxjwan |
feat(RingTheory): isotypic components |
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
new-contributor
merge-conflict
|
308/0 |
Mathlib/Order/CompactlyGenerated/Basic.lean,Mathlib/RingTheory/Isotypic.lean,Mathlib/RingTheory/SimpleModule.lean |
3 |
1 |
['github-actions'] |
nobody |
39-3576 1 month ago |
39-3576 1 month ago |
20-16585 20 days |
17246 |
pechersky author:pechersky |
feat(RingTheory/PrimaryDecomposition): PIR of Noetherian under jacobson condition |
---
- [x] depends on: #17634
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
merge-conflict
awaiting-author
|
653/1 |
Mathlib.lean,Mathlib/NumberTheory/KummerDedekind.lean,Mathlib/RingTheory/Ideal/Maps.lean,Mathlib/RingTheory/Ideal/Operations.lean,Mathlib/RingTheory/Ideal/Quotient/Operations.lean,Mathlib/RingTheory/Jacobson/Ideal.lean,Mathlib/RingTheory/PrimaryDecomposition.lean,docs/references.bib |
8 |
8 |
['erdOne', 'github-actions', 'mathlib4-dependent-issues-bot'] |
erdOne assignee:erdOne |
39-3570 1 month ago |
39-3570 1 month ago |
13-7138 13 days |
12744 |
chrisflav author:chrisflav |
feat(RingTheory/Smooth): Noetherian ring of definition |
We show that given a smooth `A`-algebra `B`, there exists a subring `A₀` of `A` of finite type over `ℤ` and a smooth `A₀`-algebra `B₀` such that `B = A ⊗[A₀] B₀`.
A reference is https://stacks.math.columbia.edu/tag/00TP.
This is also a test case for the ring of definition API.
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
merge-conflict
|
1212/0 |
Mathlib/Algebra/Algebra/Hom.lean,Mathlib/Algebra/MvPolynomial/Basic.lean,Mathlib/RingTheory/FiniteType.lean,Mathlib/RingTheory/Ideal/Operations.lean,Mathlib/RingTheory/MvPolynomial/Homogeneous.lean,Mathlib/RingTheory/RingOfDefinition/BaseChange.lean,Mathlib/RingTheory/RingOfDefinition/Basic.lean,Mathlib/RingTheory/RingOfDefinition/Relations.lean,Mathlib/RingTheory/Smooth/Descent.lean,Mathlib/ToBeMoved.lean |
10 |
0 |
[] |
nobody |
39-3545 1 month ago |
39-3545 1 month ago |
0-0 0 seconds |
12743 |
chrisflav author:chrisflav |
feat(RingTheory/RingOfDefinition): basic API |
Given a finitely presented algebra `A` over a ring `R`, we may
descend to a Noetherian subring `R₀` of `R` and a model of `A` over `R₀`.
In this PR we provide basic API for working with polynomial rings over subrings. In particular
we provide infrastructure for producing `R₀` and descending polynomials
in `R` to polynomials in `R₀` given containment of the coefficients.
Notation: `R` is a ring, `R₀` a subring, `p : MvPolynomial ι R` and `s : Set (MvPolynomial ι R)`.
## Main definitions
For producing subrings containing a set of polynomials of interest, we provide the following:
- `HasCoefficients p R₀`: typeclass expressing that the coefficients of `p` are contained in `R₀`.
- `core s`: adjoin the coefficients of a set of polynomials `s` to `ℤ`.
- `adjoinCoefficients s R₀`: adjoin the coefficients of a set of polynomials `s` to `R₀`.
- `repr p R₀`: Given `[HasCoefficients p R₀]` and a polynomial `p`, this is the representative of
`p` as a polynomial over `R₀`.
Instances for `HasCoefficients` are provided to ensure that the following facts are automatically
inferred:
- the coefficients of any polynomial in `s` are contained in `core s`.
- if the coefficients of `p` are in `R₀` and we adjoin the coefficients of `s`,
then the coefficients of `p` are also in `adjoinCoefficients s R₀`.
Now, given a (finitely) presented `R` algebra, expressed through an ideal `I : Ideal R`, a `Model`
of `I` is a structure containing
- a set `s` of generators of `I`
- a subring `R₀`
- a proof that the coefficients of `s` are contained in `R₀`
Given such a model `M`, we expose:
- `M.s₀`: the intersection of `s` with `MvPolynomial ι R₀`. Informally this is simply `s`.
- `M.I₀`: the ideal generated by `M.s₀`
- `M.A₀`: the quotient `MvPolynomial ι M.R₀ ⧸ MvPolynomial ι M.I₀`
In `RingOfDefinition/BaseChange` we show that `R ⊗[R₀] M.A₀` is `R`-isomorphic to
`MvPolynomial ι R ⧸ I` (this is done in a more general setting and then specialized
to this situation).
Since `M.I₀` is not equal to `I` intersected with `R₀`, more technical difficulties arise.
To work around these, we introduce
- `Relation A`: For an arbitrary `A : Set R`, this is simply `MvPolynomial A R`. In the following
we are particularly interested in the case where `A = s = Set (MvPolynomial ι R)` is a
set of generators of `I`.
An equation `x = y` in `MvPolynomial ι R ⧸ I` can be expressed as `x - y ∈ I`. In this case
there exists a `r : Relation s` such that `eval r = x - y`. Here `eval` is a shortcut
for `MvPolynomial.eval Subtype.val`, i.e. we evaluate the formal expression `r` in the ring
`MvPolynomial ι R`.
To preserve this equation in `MvPolynomial ι R₀ ⧸ I₀`, we need to adjoin the coefficients
of `r` to `R₀`. For this a similar API is provided, in particular:
- `HasRelation r R₀`: a typeclass expressing that the coefficients of `r` are contained in `R₀`.
- `adjoinRelations rs R₀`: adjoin the coefficients of a set of relations to `R₀`.
- `repr r M`: Given `[HasRelation r M.R₀]`, this is the representative of `r` over `R₀`, i.e.
an element of `Relation M.s₀` that is mapped to `r` under the canonical map
`Relation M.s₀ → Relation M.s`.
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
merge-conflict
|
797/0 |
Mathlib/Algebra/Algebra/Hom.lean,Mathlib/Algebra/MvPolynomial/Basic.lean,Mathlib/RingTheory/FiniteType.lean,Mathlib/RingTheory/Ideal/Operations.lean,Mathlib/RingTheory/MvPolynomial/Homogeneous.lean,Mathlib/RingTheory/RingOfDefinition/BaseChange.lean,Mathlib/RingTheory/RingOfDefinition/Basic.lean |
7 |
0 |
[] |
nobody |
39-3537 1 month ago |
39-3537 1 month ago |
0-0 0 seconds |
12695 |
chrisflav author:chrisflav |
feat(RingTheory/Smooth): smooth morphisms are flat |
We show that smooth ring homomorphisms are flat. The strategy for a smooth `A`-algebra `B` is the following:
- first we find a model of `B` over a Noetherian base ring
- if `A` is Noetherian, we identify `B` as a retract of the adic completion of a polynomial ring over `A`, which is flat
This is the summary PR which will be split in several parts.
Co-authored-by: Judith Ludwig
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
merge-conflict
|
2767/1 |
Mathlib.lean,Mathlib/Algebra/DirectSum/Basic.lean,Mathlib/Algebra/Exact.lean,Mathlib/Algebra/Module/Torsion.lean,Mathlib/LinearAlgebra/SModEq.lean,Mathlib/RingTheory/AdicCompletion/Algebra.lean,Mathlib/RingTheory/AdicCompletion/AsTensorProduct.lean,Mathlib/RingTheory/AdicCompletion/Basic.lean,Mathlib/RingTheory/AdicCompletion/Exactness.lean,Mathlib/RingTheory/AdicCompletion/Functoriality.lean,Mathlib/RingTheory/RingOfDefinition.lean,Mathlib/RingTheory/RingOfDefinition/RingModel.lean,Mathlib/RingTheory/RingOfDefinition/Utils.lean,Mathlib/RingTheory/RingOfDefinitionIdeal.lean,Mathlib/RingTheory/Smooth/Descent.lean,Mathlib/RingTheory/Smooth/Flat.lean |
16 |
0 |
[] |
nobody |
39-3529 1 month ago |
39-3529 1 month ago |
0-0 0 seconds |
12294 |
AntoineChambert-Loir author:AntoineChambert-Loir |
feat(Mathlib.RingTheory.TensorProduct.Polynomial) : tensor product of a (univariate) polynomial ring |
We define a linear equivalence of a polynomial ring by a module with a finsupp type.
We prove lemmas that allow to manipulate this equivalence.
This is adapted from the content of #12293, but since
`Polynomial` is a structure containing a `Finsupp`, these functions
can't be applied directly to `Polynomial`.
Some linear equivs need to be added to mathlib for that.
---
- [x] depends on: #12293
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
merge-conflict
WIP
|
484/0 |
Mathlib.lean,Mathlib/Algebra/MvPolynomial/Basic.lean,Mathlib/Algebra/Polynomial/Basic.lean,Mathlib/Data/Finsupp/Defs.lean,Mathlib/LinearAlgebra/TensorProduct/Tower.lean,Mathlib/RingTheory/TensorProduct/MvPolynomial.lean,Mathlib/RingTheory/TensorProduct/Polynomial.lean |
7 |
1 |
['leanprover-community-mathlib4-bot'] |
nobody |
39-3522 1 month ago |
39-3522 1 month ago |
0-79429 22 hours |
21474 |
erdOne author:erdOne |
feat(RingTheory): replace `Ring.DimensionLEOne` with `Ring.KrullDimLE` |
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
large-import
merge-conflict
|
285/170 |
Mathlib.lean,Mathlib/RingTheory/DedekindDomain/Basic.lean,Mathlib/RingTheory/DedekindDomain/Dvr.lean,Mathlib/RingTheory/DedekindDomain/Ideal.lean,Mathlib/RingTheory/DiscreteValuationRing/TFAE.lean,Mathlib/RingTheory/Ideal/Over.lean,Mathlib/RingTheory/KrullDimension/Basic.lean,Mathlib/RingTheory/KrullDimension/Localization.lean,Mathlib/RingTheory/KrullDimension/Polynomial.lean,Mathlib/RingTheory/KrullDimension/Quotient.lean,Mathlib/RingTheory/LocalRing/ResidueField/Basic.lean,Mathlib/RingTheory/Nilpotent/End.lean,Mathlib/RingTheory/Nilpotent/Lemmas.lean,Mathlib/RingTheory/PID/Quotient.lean,Mathlib/RingTheory/PrincipalIdealDomain.lean,Mathlib/RingTheory/Spectrum/Maximal/Localization.lean |
16 |
1 |
['github-actions'] |
nobody |
39-3514 1 month ago |
39-3514 1 month ago |
2-7106 2 days |
12292 |
AntoineChambert-Loir author:AntoineChambert-Loir |
feat(Mathlib.RingTheory.TensorProduct.MonoidAlgebra) : tensor product of a monoid algebra |
* `MonoidAlgebra.rTensorAlgEquiv`: the tensor product of `MonoidAlgebra M α` with `N` is `R`-linearly equivalent to `MonoidAlgebra (M ⊗[R] N) α`
* `MonoidAlgebra.scalarRTensorAlgEquiv`, the tensor product of `MonoidAlgebra R α` with `N` is `R`-linearly equivalent to `MonoidAlgebra N α`
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
merge-conflict
WIP
|
447/0 |
Mathlib.lean,Mathlib/Data/Finsupp/Defs.lean,Mathlib/RingTheory/TensorProduct/MonoidAlgebra.lean |
3 |
23 |
['AntoineChambert-Loir', 'eric-wieser', 'github-actions'] |
nobody |
39-3491 1 month ago |
39-3491 1 month ago |
6-28213 6 days |
11575 |
ScottCarnahan author:ScottCarnahan |
feat (RingTheory/HahnSeries/Addition): Lemmas on leading terms |
The main result of this PR is that when the exponent set is linearly ordered, then removing the leading term in a Hahn series `x` yields a Hahn series `y` that is, if nonzero, of strictly higher order.
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
merge-conflict
WIP
|
39/0 |
Mathlib/RingTheory/HahnSeries/Addition.lean |
1 |
0 |
[] |
nobody |
39-3484 1 month ago |
39-3484 1 month ago |
10-75677 10 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-ring-theory
merge-conflict
|
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 |
3 |
['github-actions', 'leanprover-community-bot-assistant'] |
nobody |
39-3477 1 month ago |
39-3477 1 month ago |
172-57747 172 days |
9339 |
FMLJohn author:FMLJohn |
feat (RingTheory/GradedAlgebra/HomogeneousIdeal): given a finitely generated homogeneous ideal of a graded semiring, construct a finite spanning set for the ideal which only contains homogeneous elements |
---
- [ ] depends on: #8187
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
merge-conflict
|
402/4 |
Mathlib.lean,Mathlib/Algebra/DirectSum/Internal.lean,Mathlib/Algebra/GradedMonoid.lean,Mathlib/Algebra/Module/GradeZeroModule.lean,Mathlib/RingTheory/Finiteness.lean,Mathlib/RingTheory/GradedAlgebra/Basic.lean,Mathlib/RingTheory/GradedAlgebra/HomogeneousIdeal.lean,Mathlib/RingTheory/GradedAlgebra/Noetherian.lean |
8 |
11 |
['FMLJohn', 'github-actions', 'jjaassoonn', 'leanprover-community-mathlib4-bot'] |
nobody |
39-3470 1 month ago |
39-3470 1 month ago |
0-0 0 seconds |
8195 |
newell author:newell |
feat: add a group presentation of the `DihedralGroup n` |
Add group presentation $\< a, b\ |\ a ^ 2 = 1, b ^ 2 = 1, (a * b) ^ n = 1 \>$ for `DihedralGroup n`.
---
[](https://gitpod.io/from-referrer/)
|
t-group-theory
merge-conflict
WIP
|
206/2 |
Mathlib/GroupTheory/PresentedGroup.lean,Mathlib/GroupTheory/SpecificGroups/Dihedral.lean |
2 |
6 |
['kbuzzard', 'newell'] |
nobody |
39-3313 1 month ago |
39-3313 1 month ago |
0-0 0 seconds |
11212 |
shuxuezhuyi author:shuxuezhuyi |
feat(GroupTheory/GroupAction): instance `MulAction (β ⧸ H) α` |
We instance this naturally from `MulAction β α` when `H` is a normal subgroup and acts trivially on `α`.
We also instance `IsometricSMul (M ⧸ N) X` in this way.
---
[](https://gitpod.io/from-referrer/)
|
t-group-theory
large-import
merge-conflict
awaiting-author
|
53/1 |
Mathlib/GroupTheory/GroupAction/Quotient.lean,Mathlib/Topology/MetricSpace/IsometricSMul.lean |
2 |
6 |
['YaelDillies', 'github-actions', 'grunweg', 'urkud'] |
eric-wieser assignee:eric-wieser |
39-3306 1 month ago |
39-3306 1 month ago |
193-70524 193 days |
23383 |
vlad902 author:vlad902 |
feat(GroupTheory): finitely generated groups are quotients of free groups on finite generators |
This is equivalent to the formulation that finitely generated groups/monoids are quotients of FreeGroups/Monoids over the same generators, though I think the phrasing as a surjective homomorphism is more useful. |
t-group-theory
merge-conflict
|
29/0 |
Mathlib/GroupTheory/Finiteness.lean |
1 |
1 |
['github-actions'] |
nobody |
39-3300 1 month ago |
39-3300 1 month ago |
0-0 0 seconds |
27886 |
alreadydone author:alreadydone |
feat(Algebra): (Mv)Polynomial.X is irreducible assuming NoZeroDivisors |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
awaiting-author
label:t-algebra$ |
178/66 |
Archive/Examples/Eisenstein.lean,Mathlib/Algebra/MvPolynomial/Basic.lean,Mathlib/Algebra/Polynomial/Basic.lean,Mathlib/Algebra/Polynomial/Degree/Domain.lean,Mathlib/Algebra/Polynomial/Degree/Units.lean,Mathlib/Algebra/Polynomial/Monic.lean,Mathlib/Algebra/Polynomial/RingDivision.lean,Mathlib/Combinatorics/Nullstellensatz.lean,Mathlib/RingTheory/MvPolynomial/Groebner.lean,Mathlib/RingTheory/MvPolynomial/MonomialOrder.lean,Mathlib/RingTheory/MvPolynomial/MonomialOrder/DegLex.lean,Mathlib/RingTheory/Polynomial/Content.lean,Mathlib/RingTheory/Polynomial/Eisenstein/Criterion.lean |
13 |
3 |
['alreadydone', 'github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
39-1041 1 month ago |
39-1042 1 month ago |
1-36700 1 day |
21847 |
smmercuri author:smmercuri |
feat: `v.adicCompletionIntegers K` is compact |
---
- [ ] depends on: #21844
- [ ] depends on: #24872
[](https://gitpod.io/from-referrer/)
|
large-import
t-number-theory
merge-conflict
WIP
|
459/4 |
Mathlib.lean,Mathlib/Algebra/Order/GroupWithZero/Canonical.lean,Mathlib/NumberTheory/NumberField/AdeleRing.lean,Mathlib/RingTheory/DedekindDomain/AdicValuation.lean,Mathlib/RingTheory/DedekindDomain/FiniteAdeleRing.lean,Mathlib/RingTheory/Ideal/Quotient/Basic.lean,Mathlib/Topology/Algebra/Group/Basic.lean,Mathlib/Topology/Algebra/UniformRing.lean,Mathlib/Topology/Algebra/Valued/LocallyCompact.lean,Mathlib/Topology/Algebra/Valued/ValuationTopology.lean,Mathlib/Topology/Algebra/Valued/WithZeroMulInt.lean |
11 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
38-85632 1 month ago |
38-85634 1 month ago |
0-0 0 seconds |
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
merge-conflict
|
68/8 |
.github/build.in.yml,.github/workflows/bors.yml,.github/workflows/build.yml,.github/workflows/build_fork.yml |
4 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
38-38908 1 month ago |
38-38908 1 month ago |
46-52210 46 days |
17469 |
joelriou author:joelriou |
feat(Algebra/ModuleCat/Differentials/Presheaf): the presheaf of relative differentials |
Given a functor `F : C ⥤ D`, presheaves of commutative rings `S`, `R` and a morphism `φ : S ⟶ F.op ⋙ R`, we show that derivations relative to `φ` are representable by a presheaf of `R`-modules.
This is obtained by reducing to the case of absolute differentials. The construction shall allow to deduce the presheaf version of the cokernel sequence $$f^\star \Omega_{Y/S} ⟶ \Omega_{X/S} ⟶ \Omega_{X/Y} ⟶ 0$$ when `f : X ⟶ Y` and `g : Y ⟶ S` are morphisms of schemes.
---
- [x] depends on: #17366
- [x] depends on: #19507
- [x] depends on: #17388
- [x] depends on: #16755
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebraic-geometry
t-category-theory
merge-conflict
WIP
|
391/10 |
Mathlib/Algebra/Category/ModuleCat/Differentials/Presheaf.lean |
1 |
4 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
38-34257 1 month ago |
38-34258 1 month ago |
0-530 8 minutes |
18254 |
callesonne author:callesonne |
feat(Bicategory/Modification/Pseudo): define modifications between strong natural transformations of pseudofunctors |
This PR adds modifications between strong natural transformations of pseudofunctors. At the same time, it improves the existing code on modifications between oplax natural tranformations of oplax functors (by removing some simp lemmas).
---
- [x] depends on: #18250
- [x] depends on: #18252
- [x] depends on: #18253
[](https://gitpod.io/from-referrer/)
|
t-category-theory
merge-conflict
awaiting-author
|
335/55 |
Mathlib.lean,Mathlib/CategoryTheory/Bicategory/Modification/Oplax.lean,Mathlib/CategoryTheory/Bicategory/Modification/Pseudo.lean,Mathlib/CategoryTheory/Bicategory/NaturalTransformation/Oplax.lean,Mathlib/CategoryTheory/Bicategory/NaturalTransformation/Pseudo.lean |
5 |
26 |
['callesonne', 'github-actions', 'joelriou', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'robin-carlier', 'yuma-mizuno'] |
nobody |
38-34256 1 month ago |
38-34257 1 month ago |
36-5602 36 days |
24620 |
mattrobball author:mattrobball |
chore(CategoryTheory.Basic): change `aesop_cat`'s intro transparency level to `instances` from `default` |
Let's see if this helps much.
---
[](https://gitpod.io/from-referrer/)
|
t-category-theory
merge-conflict
|
93/88 |
Mathlib/Algebra/Homology/HomologicalComplex.lean,Mathlib/Algebra/Homology/Homotopy.lean,Mathlib/Algebra/Homology/ShortComplex/Preadditive.lean,Mathlib/Algebra/Homology/Single.lean,Mathlib/CategoryTheory/Abelian/GrothendieckCategory/ModuleEmbedding/GabrielPopescu.lean,Mathlib/CategoryTheory/Adjunction/Comma.lean,Mathlib/CategoryTheory/Adjunction/Mates.lean,Mathlib/CategoryTheory/Bicategory/LocallyDiscrete.lean,Mathlib/CategoryTheory/Category/Basic.lean,Mathlib/CategoryTheory/Category/GaloisConnection.lean,Mathlib/CategoryTheory/CodiscreteCategory.lean,Mathlib/CategoryTheory/CommSq.lean,Mathlib/CategoryTheory/Comma/Over/Pullback.lean,Mathlib/CategoryTheory/Discrete/Basic.lean,Mathlib/CategoryTheory/EssentiallySmall.lean,Mathlib/CategoryTheory/FintypeCat.lean,Mathlib/CategoryTheory/Functor/EpiMono.lean,Mathlib/CategoryTheory/Functor/FullyFaithful.lean,Mathlib/CategoryTheory/Functor/KanExtension/Basic.lean,Mathlib/CategoryTheory/HomCongr.lean,Mathlib/CategoryTheory/Iso.lean,Mathlib/CategoryTheory/LiftingProperties/Adjunction.lean,Mathlib/CategoryTheory/Limits/ConeCategory.lean,Mathlib/CategoryTheory/Limits/HasLimits.lean,Mathlib/CategoryTheory/Limits/IsLimit.lean,Mathlib/CategoryTheory/Limits/Preserves/Shapes/Terminal.lean,Mathlib/CategoryTheory/Limits/Shapes/ZeroMorphisms.lean,Mathlib/CategoryTheory/MorphismProperty/OverAdjunction.lean,Mathlib/CategoryTheory/Preadditive/Opposite.lean,Mathlib/CategoryTheory/SingleObj.lean,Mathlib/Topology/Sheaves/Sheaf.lean |
31 |
8 |
['github-actions', 'leanprover-bot', 'mathlib4-merge-conflict-bot', 'mattrobball'] |
nobody |
38-25061 1 month ago |
38-25061 1 month ago |
0-0 0 seconds |
25288 |
robertmaxton42 author:robertmaxton42 |
feat(CategoryTheory): generalize `Discrete` to arbitrary morphism levels |
Using an unused `let`, add an 'anchor' to the definition of `Discrete`, allowing it to carry a second universe level that is then used to permit discrete categories to live in any `Cat.{v, u}`. (This trick was borrowed from the code of `ULiftHom`.)
---
[](https://gitpod.io/from-referrer/)
|
t-category-theory
merge-conflict
|
38/32 |
Mathlib/CategoryTheory/Bicategory/LocallyDiscrete.lean,Mathlib/CategoryTheory/Discrete/Basic.lean,Mathlib/CategoryTheory/IsConnected.lean |
3 |
3 |
['github-actions', 'joelriou', 'mathlib4-merge-conflict-bot'] |
nobody |
38-23616 1 month ago |
38-23617 1 month ago |
0-0 0 seconds |
27709 |
kckennylau author:kckennylau |
chore: fix links |
---
See https://github.com/leanprover-community/mathlib4/pull/27545#discussion_r2238206933
[](https://gitpod.io/from-referrer/)
|
merge-conflict
WIP
|
269/256 |
Mathlib/Algebra/Algebra/Bilinear.lean,Mathlib/Algebra/GCDMonoid/Multiset.lean,Mathlib/Algebra/Group/Even.lean,Mathlib/Algebra/Group/Pi/Basic.lean,Mathlib/Algebra/Group/Pi/Lemmas.lean,Mathlib/Algebra/Group/TypeTags/Basic.lean,Mathlib/Algebra/Homology/DerivedCategory/Basic.lean,Mathlib/Algebra/Homology/Embedding/Basic.lean,Mathlib/Algebra/Module/Hom.lean,Mathlib/Algebra/Module/Submodule/Bilinear.lean,Mathlib/Algebra/Order/Field/Pi.lean,Mathlib/Algebra/Order/GroupWithZero/Unbundled/Basic.lean,Mathlib/Algebra/Order/Hom/Basic.lean,Mathlib/Algebra/Order/Monovary.lean,Mathlib/Algebra/Order/Ring/Unbundled/Basic.lean,Mathlib/Algebra/Order/Ring/Unbundled/Rat.lean,Mathlib/Algebra/Ring/Basic.lean,Mathlib/Algebra/Squarefree/Basic.lean,Mathlib/Algebra/Star/BigOperators.lean,Mathlib/Algebra/Star/Free.lean,Mathlib/Algebra/Star/SelfAdjoint.lean,Mathlib/Analysis/Analytic/RadiusLiminf.lean,Mathlib/Analysis/CStarAlgebra/Matrix.lean,Mathlib/Analysis/Calculus/Conformal/NormedSpace.lean,Mathlib/Analysis/Calculus/Deriv/Add.lean,Mathlib/Analysis/Calculus/Deriv/Inv.lean,Mathlib/Analysis/Calculus/Deriv/Inverse.lean,Mathlib/Analysis/Calculus/Deriv/Linear.lean,Mathlib/Analysis/Calculus/Deriv/Mul.lean,Mathlib/Analysis/Complex/Basic.lean,Mathlib/Analysis/Complex/Circle.lean,Mathlib/Analysis/Complex/OperatorNorm.lean,Mathlib/Analysis/Convex/Function.lean,Mathlib/Analysis/Convex/Jensen.lean,Mathlib/Analysis/Meromorphic/IsolatedZeros.lean,Mathlib/Analysis/Normed/Operator/BoundedLinearMaps.lean,Mathlib/Analysis/SpecialFunctions/Exponential.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Basic.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Bounds.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/EulerSineProd.lean,Mathlib/CategoryTheory/Abelian/Opposite.lean,Mathlib/CategoryTheory/Adjunction/Opposites.lean,Mathlib/CategoryTheory/Bicategory/Functor/Pseudofunctor.lean,Mathlib/CategoryTheory/Closed/Monoidal.lean,Mathlib/CategoryTheory/Limits/Shapes/Kernels.lean,Mathlib/CategoryTheory/Localization/Equivalence.lean,Mathlib/CategoryTheory/Localization/Trifunctor.lean,Mathlib/CategoryTheory/ObjectProperty/Basic.lean,Mathlib/CategoryTheory/Sites/Coherent/SheafComparison.lean,Mathlib/Combinatorics/Colex.lean,Mathlib/Combinatorics/Hall/Finite.lean,Mathlib/Combinatorics/Pigeonhole.lean,Mathlib/Combinatorics/Quiver/Covering.lean,Mathlib/Combinatorics/Quiver/Path.lean,Mathlib/Control/LawfulFix.lean,Mathlib/Data/Complex/Basic.lean,Mathlib/Data/Fin/Pigeonhole.lean,Mathlib/Data/FinEnum/Option.lean,Mathlib/Data/Finset/Filter.lean,Mathlib/Data/Finsupp/Fin.lean,Mathlib/Data/Fintype/BigOperators.lean,Mathlib/Data/Fintype/Defs.lean,Mathlib/Data/Int/Basic.lean,Mathlib/Data/Int/Cast/Basic.lean,Mathlib/Data/Int/Cast/Lemmas.lean,Mathlib/Data/Int/Lemmas.lean,Mathlib/Data/Int/Order/Lemmas.lean,Mathlib/Data/Int/Range.lean,Mathlib/Data/List/Chain.lean,Mathlib/Data/List/Dedup.lean,Mathlib/Data/List/Destutter.lean,Mathlib/Data/List/Forall2.lean,Mathlib/Data/List/Lattice.lean,Mathlib/Data/List/Lemmas.lean,Mathlib/Data/List/Nodup.lean,Mathlib/Data/List/Pairwise.lean,Mathlib/Data/List/Permutation.lean,Mathlib/Data/List/ProdSigma.lean,Mathlib/Data/List/Sections.lean,Mathlib/Data/List/Sublists.lean,Mathlib/Data/Matrix/Notation.lean,Mathlib/Data/Matroid/Minor/Restrict.lean,Mathlib/Data/Multiset/FinsetOps.lean,Mathlib/Data/Nat/Basic.lean,Mathlib/Data/Nat/Cast/WithTop.lean,Mathlib/Data/Nat/Choose/Basic.lean,Mathlib/Data/Nat/Factorization/Basic.lean,Mathlib/Data/Nat/Factorization/LCM.lean,Mathlib/Data/PSigma/Order.lean,Mathlib/Data/Prod/Lex.lean,Mathlib/Data/Rat/Encodable.lean,Mathlib/Data/Set/Card.lean,Mathlib/Data/Set/Defs.lean,Mathlib/Data/Set/Finite/Basic.lean,Mathlib/Data/Set/Finite/Lattice.lean,Mathlib/Data/Set/Functor.lean,Mathlib/Data/Set/Notation.lean,Mathlib/Data/Set/Pairwise/Basic.lean,Mathlib/Data/Set/Prod.lean,Mathlib/Data/Sigma/Lex.lean |
157 |
87 |
['github-actions', 'kbuzzard', 'kckennylau', 'mathlib4-merge-conflict-bot'] |
nobody |
38-21827 1 month ago |
38-21827 1 month ago |
0-9 9 seconds |
10345 |
newell author:newell |
feat(Algebra.Module.Zlattice): Add Voronoi Domain |
Adds the definition for a Voronoi Domain in regards to the $\mathbb{Z}$-lattice:
$$C := \lbrace\mathbf{w} \in \mathbb{V}^n\ :\ |\mathbf{w}| \leq |\mathbf{w} - \mathbf{v}|\ \text{for all}\ \mathbf{v} \in \mathbf{L} \rbrace$$
where $\mathbf{L}\$ is the $\mathbb{Z}$-lattice.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
WIP
label:t-algebra$ |
17/0 |
Mathlib/Algebra/Module/Zlattice.lean |
1 |
3 |
['alreadydone', 'newell'] |
nobody |
37-39715 1 month ago |
37-39715 1 month ago |
0-0 0 seconds |
27286 |
edegeltje author:edegeltje |
refactor(OrderDual): make a one-field structure and remove defeq abuse |
---
[](https://gitpod.io/from-referrer/)
|
t-order
merge-conflict
WIP
|
683/426 |
Mathlib/Algebra/Field/Basic.lean,Mathlib/Algebra/Order/Group/Action/Synonym.lean,Mathlib/Algebra/Order/Group/Synonym.lean,Mathlib/Algebra/Order/GroupWithZero/Action/Synonym.lean,Mathlib/Algebra/Order/GroupWithZero/Synonym.lean,Mathlib/Algebra/Order/Module/Synonym.lean,Mathlib/Algebra/Order/Monoid/Unbundled/OrderDual.lean,Mathlib/Algebra/Order/Ring/Synonym.lean,Mathlib/Data/Nat/Cast/Synonym.lean,Mathlib/Logic/Function/Iterate.lean,Mathlib/Order/Basic.lean,Mathlib/Order/BoundedOrder/Basic.lean,Mathlib/Order/BoundedOrder/Lattice.lean,Mathlib/Order/BoundedOrder/Monotone.lean,Mathlib/Order/Circular.lean,Mathlib/Order/Compare.lean,Mathlib/Order/Disjoint.lean,Mathlib/Order/GaloisConnection/Defs.lean,Mathlib/Order/Iterate.lean,Mathlib/Order/Lattice.lean,Mathlib/Order/Max.lean,Mathlib/Order/MinMax.lean,Mathlib/Order/Monotone/Basic.lean,Mathlib/Order/RelClasses.lean,Mathlib/Order/Synonym.lean,Mathlib/Order/WithBot.lean |
26 |
2 |
['alreadydone', 'github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
37-39437 1 month ago |
37-39438 1 month ago |
0-0 0 seconds |
27950 |
alreadydone author:alreadydone |
feat(MonoidAlgebra): criteria for `single` to be a unit, irreducible or prime |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
WIP
label:t-algebra$ |
714/192 |
Mathlib.lean,Mathlib/Algebra/BigOperators/Group/Finset/Basic.lean,Mathlib/Algebra/BigOperators/Group/Finset/Defs.lean,Mathlib/Algebra/BigOperators/Group/Finset/Piecewise.lean,Mathlib/Algebra/BigOperators/Group/List/Lemmas.lean,Mathlib/Algebra/BigOperators/Group/Multiset/Basic.lean,Mathlib/Algebra/Divisibility/Basic.lean,Mathlib/Algebra/Divisibility/Finite.lean,Mathlib/Algebra/Divisibility/Hom.lean,Mathlib/Algebra/Divisibility/Prod.lean,Mathlib/Algebra/Divisibility/Units.lean,Mathlib/Algebra/Group/Action/Pointwise/Finset.lean,Mathlib/Algebra/Group/Irreducible/Lemmas.lean,Mathlib/Algebra/Group/Prod.lean,Mathlib/Algebra/GroupWithZero/Associated.lean,Mathlib/Algebra/MonoidAlgebra/Divisibility.lean,Mathlib/Algebra/MonoidAlgebra/NoZeroDivisors.lean,Mathlib/Algebra/Notation/Defs.lean,Mathlib/Algebra/Prime/Defs.lean,Mathlib/Algebra/Prime/Lemmas.lean,Mathlib/Algebra/Prime/Prod.lean,Mathlib/Data/Nat/Init.lean,Mathlib/Dynamics/PeriodicPts/Defs.lean,Mathlib/GroupTheory/Coset/Card.lean,Mathlib/GroupTheory/Exponent.lean,Mathlib/GroupTheory/GroupAction/Blocks.lean,Mathlib/GroupTheory/GroupAction/Period.lean,Mathlib/GroupTheory/Index.lean,Mathlib/GroupTheory/OrderOfElement.lean,Mathlib/GroupTheory/Perm/Cycle/Type.lean,Mathlib/GroupTheory/Schreier.lean,Mathlib/GroupTheory/SpecificGroups/Cyclic.lean,Mathlib/Tactic/ToAdditive/Frontend.lean |
33 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
37-38901 1 month ago |
37-38902 1 month ago |
0-53 53 seconds |
27378 |
peakpoint author:peakpoint |
refactor(Geometry/Euclidean/Projection): redefine projection and reflection for affine subspaces |
This PR continues the work from #25578.
Original PR: https://github.com/leanprover-community/mathlib4/pull/25578 |
new-contributor
t-euclidean-geometry
merge-conflict
|
316/317 |
Mathlib/Analysis/Normed/Affine/ContinuousAffineMap.lean,Mathlib/Analysis/Normed/Affine/Isometry.lean,Mathlib/Geometry/Euclidean/Circumcenter.lean,Mathlib/Geometry/Euclidean/Projection.lean |
4 |
7 |
['github-actions', 'jsm28', 'leanprover-community-bot-assistant', 'mathlib4-merge-conflict-bot', 'peakpoint'] |
nobody |
35-64118 1 month ago |
35-64119 1 month ago |
15-31164 15 days |
20671 |
thefundamentaltheor3m author:thefundamentaltheor3m |
feat(Analysis/Asymptotics/SpecificAsymptotics): Proving that 𝛔ₖ(n) = O(nᵏ⁺¹) |
This PR proves a result about the $\sigma_k(n)$ arithmetic function, namely, that it is $O\left(n^{k+1}\right)$. Main theorem:
`theorem sigma_asymptotic (k : ℕ) : (fun n ↦ (σ k n : ℝ)) =O[atTop] (fun n ↦ (n ^ (k + 1) : ℝ))`
This result was proved as part of the sphere packing project.
---
[](https://gitpod.io/from-referrer/)
|
large-import
new-contributor
t-number-theory
merge-conflict
awaiting-author
|
29/0 |
Mathlib/Analysis/Asymptotics/SpecificAsymptotics.lean |
1 |
3 |
['b-mehta', 'github-actions', 'mathlib4-merge-conflict-bot'] |
b-mehta assignee:b-mehta |
34-7117 1 month ago |
34-7117 1 month ago |
9-59130 9 days |
20267 |
joelriou author:joelriou |
feat(CategoryTheory): comma categories are accessible |
---
(I shall probably not work on this PR in the near future.)
- [ ] depends on: #19937
- [ ] depends on: #19945
- [ ] depends on: #19959
- [ ] depends on: #20005
- [ ] depends on: #19955
- [x] depends on: #20263
[](https://gitpod.io/from-referrer/)
|
t-category-theory
merge-conflict
awaiting-author
WIP
|
1513/7 |
Mathlib.lean,Mathlib/CategoryTheory/Comma/Arrow.lean,Mathlib/CategoryTheory/Comma/CardinalArrow.lean,Mathlib/CategoryTheory/EssentiallySmall.lean,Mathlib/CategoryTheory/Limits/Comma.lean,Mathlib/CategoryTheory/Limits/TypesFiltered.lean,Mathlib/CategoryTheory/Presentable/Basic.lean,Mathlib/CategoryTheory/Presentable/CardinalFilteredPresentation.lean,Mathlib/CategoryTheory/Presentable/Comma.lean,Mathlib/CategoryTheory/Presentable/IsCardinalFiltered.lean,Mathlib/CategoryTheory/Presentable/Limits.lean,Mathlib/CategoryTheory/Presentable/LocallyPresentable.lean,Mathlib/CategoryTheory/Presentable/ParallelMaps.lean,Mathlib/SetTheory/Cardinal/HasCardinalLT.lean,docs/references.bib |
15 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
34-84 1 month ago |
34-85 1 month ago |
0-0 0 seconds |
27451 |
kckennylau author:kckennylau |
feat(RingTheory/Valuation): define ball, closed ball, and sphere |
*From the 2025 Local Class Field Theory Workshop.*
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
merge-conflict
|
27/0 |
Mathlib/RingTheory/Valuation/Basic.lean |
1 |
13 |
['JovanGerb', 'github-actions', 'kckennylau', 'mathlib4-merge-conflict-bot', 'pechersky', 'wwylele'] |
nobody |
32-71411 1 month ago |
32-71412 1 month ago |
17-52359 17 days |
27987 |
kckennylau author:kckennylau |
feat(RingTheory/Valuation): define ball, closed ball, and sphere |
---
The pullback PR of #26827 and #27451.
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
large-import
merge-conflict
|
73/0 |
Mathlib/RingTheory/Valuation/Basic.lean |
1 |
4 |
['JovanGerb', 'github-actions', 'kckennylau', 'mathlib4-merge-conflict-bot'] |
nobody |
32-71040 1 month ago |
32-71041 1 month ago |
6-6455 6 days |
24862 |
grunweg author:grunweg |
feat(LocallyIntegrable): generalise more to enorms |
---
Note: github's diff is very confused; it includes changes which very clearly are already on the master branch.
I'll see which of the remaining changes after the dependencies have landed is already polished enough.
- [x] depends on: #24352
- [x] depends on: #27457 (this half is settled already)
- [ ] open question: filter lemmas; IsBoundedUnder is not the right condition as-is; need to think (or just not generalise)
[](https://gitpod.io/from-referrer/)
|
carleson
t-measure-probability
merge-conflict
WIP
|
171/88 |
Mathlib/MeasureTheory/Function/L1Space/HasFiniteIntegral.lean,Mathlib/MeasureTheory/Function/LocallyIntegrable.lean,Mathlib/MeasureTheory/Integral/IntegrableOn.lean |
3 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
32-64761 1 month ago |
32-64762 1 month ago |
0-1 1 second |
25978 |
Bergschaf author:Bergschaf |
feat(Order/Sublocale): Open Sublocales |
---
[](https://gitpod.io/from-referrer/)
- [ ] depends on: #25089 |
t-order
merge-conflict
|
377/8 |
Mathlib.lean,Mathlib/Order/Hom/Lattice.lean,Mathlib/Order/Nucleus.lean,Mathlib/Order/Sublocale.lean,Mathlib/Order/Synonym.lean,docs/references.bib |
6 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
32-16202 1 month ago |
32-16203 1 month ago |
0-1908 31 minutes |
27197 |
alreadydone author:alreadydone |
feat(Topology): `IsCoveringMapOn` open set |
---
- [x] depends on: #25044
[](https://gitpod.io/from-referrer/)
|
t-topology
merge-conflict
WIP
|
282/28 |
Mathlib/Topology/Covering.lean,Mathlib/Topology/FiberBundle/Trivialization.lean,Mathlib/Topology/Homeomorph/Lemmas.lean,Mathlib/Topology/Maps/Basic.lean |
4 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
31-78311 1 month ago |
31-79016 1 month ago |
0-0 0 seconds |
25133 |
erdOne author:erdOne |
feat(Tactic/NormNum): support positive characteristic |
Co-authored-by: Heather Macbeth
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-meta
merge-conflict
WIP
|
250/39 |
Mathlib/Tactic/NormNum/CharP.lean,Mathlib/Tactic/NormNum/Core.lean,Mathlib/Tactic/NormNum/Eq.lean,Mathlib/Tactic/NormNum/Inv.lean,Mathlib/Tactic/NormNum/Test.lean |
5 |
5 |
['erdOne', 'eric-wieser', 'github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
30-86200 30 days ago |
30-86201 30 days ago |
0-0 0 seconds |
27003 |
eric-wieser author:eric-wieser |
chore: use `Simp.ResultQ` more often |
Also uses `~q` in place of manual `isDefEq` matching.
---
[](https://gitpod.io/from-referrer/)
|
t-meta
merge-conflict
|
18/22 |
Mathlib/Tactic/NormNum/Core.lean,Mathlib/Tactic/NormNum/Result.lean,Mathlib/Tactic/ReduceModChar.lean |
3 |
7 |
['JovanGerb', 'eric-wieser', 'github-actions', 'mathlib4-merge-conflict-bot'] |
JovanGerb assignee:JovanGerb |
30-85664 30 days ago |
30-85665 30 days ago |
32-70098 32 days |
26374 |
joelriou author:joelriou |
feat(CategoryTheory): existence of right derived functors using derivability structures |
In this PR, we formalize an existence theorem for right derived functors which appeared in the article _Structures de dérivabilité_ by Bruno Kahn and Georges Maltsiniotis, Adv. Math. 218 (2008).
---
- [ ] depends on: #26036
This PR continues the work from #22508.
Original PR: https://github.com/leanprover-community/mathlib4/pull/22508 |
t-category-theory
merge-conflict
WIP
|
326/2 |
Mathlib.lean,Mathlib/CategoryTheory/Functor/Derived/PointwiseRightDerived.lean,Mathlib/CategoryTheory/Iso.lean,Mathlib/CategoryTheory/Limits/Final.lean,Mathlib/CategoryTheory/Localization/DerivabilityStructure/Basic.lean,Mathlib/CategoryTheory/Localization/DerivabilityStructure/PointwiseRightDerived.lean |
6 |
4 |
['github-actions', 'joelriou', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
30-76498 30 days ago |
30-76498 30 days ago |
0-53 53 seconds |
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
merge-conflict
|
103/0 |
Mathlib/Data/Set/Prod.lean,Mathlib/SetTheory/ZFC/Basic.lean |
2 |
10 |
['Ruben-VandeVelde', 'VTrelat', 'github-actions', 'leanprover-community-bot-assistant'] |
nobody |
30-75307 30 days ago |
70-23214 2 months ago |
29-56208 29 days |
24754 |
urkud author:urkud |
feat: define `pathIntegral` |
This is a step towards formalizing of the Poincaré lemma for 1-forms.
---
- [x] depends on: #24831
- [x] depends on: #25047
- [x] depends on: #25048
[](https://gitpod.io/from-referrer/)
|
t-analysis
merge-conflict
awaiting-author
|
552/8 |
Mathlib.lean,Mathlib/Analysis/Convex/PathConnected.lean,Mathlib/Analysis/Normed/Module/Basic.lean,Mathlib/MeasureTheory/Integral/IntervalIntegral/Basic.lean,Mathlib/MeasureTheory/Integral/PathIntegral/Basic.lean |
5 |
24 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'sgouezel', 'urkud'] |
nobody |
30-74903 30 days ago |
30-74904 30 days ago |
8-52615 8 days |
16150 |
urkud author:urkud |
feat(Dynamics): Hopf decomposition |
Prove Hopf decomposition.
- [ ] rewrite to work with the saturations right away, not with a wandering set.
- [ ] generalize to an action of a countable group, use fundamental domains.
---
- [ ] depends on: #16146
- [ ] depends on: #16126
[](https://gitpod.io/from-referrer/)
|
t-dynamics
t-measure-probability
merge-conflict
|
212/0 |
Mathlib.lean,Mathlib/Dynamics/Ergodic/Dissipative.lean,Mathlib/MeasureTheory/MeasurableSpace/Basic.lean |
3 |
4 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'urkud'] |
nobody |
30-53636 30 days ago |
30-53637 30 days ago |
0-0 0 seconds |
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
merge-conflict
|
342/0 |
Mathlib.lean,Mathlib/Util/CommandElabHook.lean,Mathlib/Util/SuppressSorry.lean,MathlibTest/suppressSorry.lean |
4 |
15 |
['digama0', 'eric-wieser', 'github-actions', 'mathlib4-merge-conflict-bot'] |
alexjbest assignee:alexjbest |
30-40460 30 days ago |
30-40460 30 days ago |
71-28549 71 days |
26394 |
winstonyin author:winstonyin |
feat: existence of local flows on manifolds |
This PR continues the work from #21777.
Original PR: https://github.com/leanprover-community/mathlib4/pull/21777
Transfer the existence theorem of local flows on vector spaces to manifolds. The precise statement is:
> If a vector field `v` on a manifold `M` is continuously differentiable at an interior point `x₀`, then for a given `t₀` there exists a neighbourhood `u` of `x₀`, a positive `ε`, and `γ : M → ℝ → M` such that `γ x` is an integral curve of `v` on `(t₀ - ε, t₀ + ε)` for all `x ∈ u`.
This is powerful because all curves `γ x` (each with initial condition `x ∈ u`) share the same existence time interval `(t₀ - ε, t₀ + ε)`, rather than each curve having its own `ε`. This will allow us to show that $C^1$ vector fields on compact manifolds always have global integral curves / global flows.
Any suggestions to shorten the proof or split out useful lemmas are welcome!
- [x] depends on: #26392
---
[](https://gitpod.io/from-referrer/)
|
t-differential-geometry
merge-conflict
WIP
|
154/52 |
Mathlib/Analysis/ODE/PicardLindelof.lean,Mathlib/Geometry/Manifold/IntegralCurve/ExistUnique.lean,Mathlib/Order/Filter/Prod.lean |
3 |
5 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'winstonyin'] |
nobody |
30-40021 30 days ago |
30-40022 30 days ago |
0-70 1 minute |
26446 |
joelriou author:joelriou |
refactor(CategoryTheory): make morphisms in full subcategories a 1-field structure |
This PR refactors the definition of morphisms in full subcategories (and induced categories), by making them a 1-field structure. This prevents certain defeq abuse, and improves automation. (The only issue is that this adds an extra layer: `f` sometimes becomes `f.hom`, etc.)
---
(This time, I will try to complete this refactor. I very much need this for application to homotopical algebra, where full subcategories of cofibrant/fibrant/bifibrant are used.)
[](https://gitpod.io/from-referrer/)
|
t-category-theory
merge-conflict
WIP
|
1741/1418 |
Mathlib/Algebra/Category/CommAlgCat/FiniteType.lean,Mathlib/Algebra/Category/FGModuleCat/Basic.lean,Mathlib/Algebra/Category/FGModuleCat/EssentiallySmall.lean,Mathlib/Algebra/Category/Grp/FiniteGrp.lean,Mathlib/Algebra/Category/Grp/LeftExactFunctor.lean,Mathlib/Algebra/Category/ModuleCat/Tannaka.lean,Mathlib/Algebra/Homology/LocalCohomology.lean,Mathlib/AlgebraicGeometry/AffineScheme.lean,Mathlib/AlgebraicGeometry/Cover/Open.lean,Mathlib/AlgebraicGeometry/FunctionField.lean,Mathlib/AlgebraicGeometry/GammaSpecAdjunction.lean,Mathlib/AlgebraicGeometry/Gluing.lean,Mathlib/AlgebraicGeometry/Morphisms/QuasiSeparated.lean,Mathlib/AlgebraicGeometry/Morphisms/Separated.lean,Mathlib/AlgebraicGeometry/Noetherian.lean,Mathlib/AlgebraicGeometry/OpenImmersion.lean,Mathlib/AlgebraicGeometry/Scheme.lean,Mathlib/AlgebraicGeometry/Spec.lean,Mathlib/AlgebraicTopology/SimplexCategory/Basic.lean,Mathlib/AlgebraicTopology/SimplexCategory/Defs.lean,Mathlib/AlgebraicTopology/SimplexCategory/MorphismProperty.lean,Mathlib/AlgebraicTopology/SimplicialNerve.lean,Mathlib/AlgebraicTopology/SimplicialSet/Coskeletal.lean,Mathlib/AlgebraicTopology/SimplicialSet/HomotopyCat.lean,Mathlib/AlgebraicTopology/SimplicialSet/NerveAdjunction.lean,Mathlib/AlgebraicTopology/SimplicialSet/Path.lean,Mathlib/CategoryTheory/Abelian/GrothendieckCategory/ColimCoyoneda.lean,Mathlib/CategoryTheory/Abelian/GrothendieckCategory/EnoughInjectives.lean,Mathlib/CategoryTheory/Abelian/GrothendieckCategory/Subobject.lean,Mathlib/CategoryTheory/Action/Concrete.lean,Mathlib/CategoryTheory/Action/Continuous.lean,Mathlib/CategoryTheory/Adjunction/PartialAdjoint.lean,Mathlib/CategoryTheory/Category/TwoP.lean,Mathlib/CategoryTheory/ConcreteCategory/Basic.lean,Mathlib/CategoryTheory/ConnectedComponents.lean,Mathlib/CategoryTheory/Countable.lean,Mathlib/CategoryTheory/Endomorphism.lean,Mathlib/CategoryTheory/EqToHom.lean,Mathlib/CategoryTheory/EssentialImage.lean,Mathlib/CategoryTheory/EssentiallySmall.lean,Mathlib/CategoryTheory/Filtered/Small.lean,Mathlib/CategoryTheory/FinCategory/AsType.lean,Mathlib/CategoryTheory/FintypeCat.lean,Mathlib/CategoryTheory/Galois/Basic.lean,Mathlib/CategoryTheory/Galois/Decomposition.lean,Mathlib/CategoryTheory/Galois/Equivalence.lean,Mathlib/CategoryTheory/Galois/EssSurj.lean,Mathlib/CategoryTheory/Galois/Examples.lean,Mathlib/CategoryTheory/Galois/GaloisObjects.lean,Mathlib/CategoryTheory/Galois/IsFundamentalgroup.lean,Mathlib/CategoryTheory/Galois/Prorepresentability.lean,Mathlib/CategoryTheory/Galois/Topology.lean,Mathlib/CategoryTheory/InducedCategory.lean,Mathlib/CategoryTheory/Limits/ExactFunctor.lean,Mathlib/CategoryTheory/Limits/Final.lean,Mathlib/CategoryTheory/Limits/Indization/LocallySmall.lean,Mathlib/CategoryTheory/Linear/Basic.lean,Mathlib/CategoryTheory/Localization/Construction.lean,Mathlib/CategoryTheory/Localization/LocallySmall.lean,Mathlib/CategoryTheory/Localization/Predicate.lean,Mathlib/CategoryTheory/Monoidal/Braided/Basic.lean,Mathlib/CategoryTheory/Monoidal/Cartesian/Basic.lean,Mathlib/CategoryTheory/Monoidal/Cartesian/Grp_.lean,Mathlib/CategoryTheory/Monoidal/Category.lean,Mathlib/CategoryTheory/Monoidal/CommGrp_.lean,Mathlib/CategoryTheory/Monoidal/CommMon_.lean,Mathlib/CategoryTheory/Monoidal/Grp_.lean,Mathlib/CategoryTheory/Monoidal/Internal/FunctorCategory.lean,Mathlib/CategoryTheory/Monoidal/Internal/Types/Basic.lean,Mathlib/CategoryTheory/Monoidal/Internal/Types/CommGrp_.lean,Mathlib/CategoryTheory/Monoidal/Internal/Types/Grp_.lean,Mathlib/CategoryTheory/Monoidal/Subcategory.lean,Mathlib/CategoryTheory/MorphismProperty/IsInvertedBy.lean,Mathlib/CategoryTheory/ObjectProperty/FullSubcategory.lean,Mathlib/CategoryTheory/Preadditive/AdditiveFunctor.lean,Mathlib/CategoryTheory/Preadditive/Basic.lean,Mathlib/CategoryTheory/Preadditive/CommGrp_.lean,Mathlib/CategoryTheory/Simple.lean,Mathlib/CategoryTheory/Sites/Coherent/RegularSheaves.lean,Mathlib/CategoryTheory/Sites/EffectiveEpimorphic.lean,Mathlib/CategoryTheory/Sites/Sheaf.lean,Mathlib/CategoryTheory/Sites/SheafHom.lean,Mathlib/CategoryTheory/Sites/SheafOfTypes.lean,Mathlib/CategoryTheory/Skeletal.lean,Mathlib/CategoryTheory/Subobject/Basic.lean,Mathlib/CategoryTheory/Subobject/Comma.lean,Mathlib/CategoryTheory/Subobject/FactorThru.lean,Mathlib/CategoryTheory/Subobject/Lattice.lean,Mathlib/CategoryTheory/Subobject/MonoOver.lean,Mathlib/CategoryTheory/Subobject/NoetherianObject.lean,Mathlib/CategoryTheory/Subobject/Types.lean,Mathlib/CategoryTheory/Subpresheaf/Subobject.lean,Mathlib/CategoryTheory/Subterminal.lean,Mathlib/CategoryTheory/Topos/Classifier.lean,Mathlib/Condensed/Discrete/Colimit.lean,Mathlib/Condensed/Discrete/LocallyConstant.lean,Mathlib/Condensed/Discrete/Module.lean,Mathlib/Condensed/Light/TopCatAdjunction.lean,Mathlib/Condensed/TopCatAdjunction.lean,Mathlib/Condensed/TopComparison.lean |
141 |
7 |
['erdOne', 'github-actions', 'joelriou', 'leanprover-community-bot-assistant', 'smorel394'] |
nobody |
30-18005 30 days ago |
49-31027 1 month ago |
0-2 2 seconds |
28298 |
thorimur author:thorimur |
chore: dedent `to_additive` docstrings |
This PR uses automation to dedent `to_additive` docstrings throughout Mathlib. It does not lint against indentation or in any way enforce indentation standards for future docstrings. The convention was chosen in accordance with the discussion and polls at [this Zulip thread](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Poll.3A.20Indentation.20style.20for.20.60to_additive.60.20docstrings/with/534285603).
---
[](https://gitpod.io/from-referrer/)
|
awaiting-zulip
merge-conflict
documentation
|
949/949 |
Mathlib/Algebra/BigOperators/Fin.lean,Mathlib/Algebra/BigOperators/Finprod.lean,Mathlib/Algebra/BigOperators/Finsupp/Basic.lean,Mathlib/Algebra/BigOperators/Group/Finset/Lemmas.lean,Mathlib/Algebra/BigOperators/Group/List/Basic.lean,Mathlib/Algebra/BigOperators/Group/Multiset/Defs.lean,Mathlib/Algebra/BigOperators/Pi.lean,Mathlib/Algebra/Category/Grp/Basic.lean,Mathlib/Algebra/Category/Grp/FilteredColimits.lean,Mathlib/Algebra/Category/Grp/Limits.lean,Mathlib/Algebra/Category/Grp/Ulift.lean,Mathlib/Algebra/Category/MonCat/Basic.lean,Mathlib/Algebra/Category/MonCat/FilteredColimits.lean,Mathlib/Algebra/Category/MonCat/Limits.lean,Mathlib/Algebra/Category/Semigrp/Basic.lean,Mathlib/Algebra/Free.lean,Mathlib/Algebra/FreeMonoid/Basic.lean,Mathlib/Algebra/Group/Action/Defs.lean,Mathlib/Algebra/Group/Action/Pi.lean,Mathlib/Algebra/Group/Action/Pointwise/Finset.lean,Mathlib/Algebra/Group/Basic.lean,Mathlib/Algebra/Group/Defs.lean,Mathlib/Algebra/Group/Embedding.lean,Mathlib/Algebra/Group/Equiv/Basic.lean,Mathlib/Algebra/Group/Equiv/Defs.lean,Mathlib/Algebra/Group/Equiv/Opposite.lean,Mathlib/Algebra/Group/Even.lean,Mathlib/Algebra/Group/Hom/Basic.lean,Mathlib/Algebra/Group/Hom/Defs.lean,Mathlib/Algebra/Group/Hom/Instances.lean,Mathlib/Algebra/Group/Indicator.lean,Mathlib/Algebra/Group/Pi/Lemmas.lean,Mathlib/Algebra/Group/Pi/Units.lean,Mathlib/Algebra/Group/Pointwise/Finset/Basic.lean,Mathlib/Algebra/Group/Pointwise/Set/Basic.lean,Mathlib/Algebra/Group/Prod.lean,Mathlib/Algebra/Group/Subgroup/Basic.lean,Mathlib/Algebra/Group/Subgroup/Defs.lean,Mathlib/Algebra/Group/Subgroup/Ker.lean,Mathlib/Algebra/Group/Subgroup/Lattice.lean,Mathlib/Algebra/Group/Subgroup/Map.lean,Mathlib/Algebra/Group/Subgroup/Pointwise.lean,Mathlib/Algebra/Group/Submonoid/Basic.lean,Mathlib/Algebra/Group/Submonoid/BigOperators.lean,Mathlib/Algebra/Group/Submonoid/Defs.lean,Mathlib/Algebra/Group/Submonoid/Membership.lean,Mathlib/Algebra/Group/Submonoid/MulAction.lean,Mathlib/Algebra/Group/Submonoid/Operations.lean,Mathlib/Algebra/Group/Subsemigroup/Basic.lean,Mathlib/Algebra/Group/Subsemigroup/Operations.lean,Mathlib/Algebra/Group/UniqueProds/Basic.lean,Mathlib/Algebra/Group/Units/Defs.lean,Mathlib/Algebra/Group/Units/Equiv.lean,Mathlib/Algebra/Group/Units/Hom.lean,Mathlib/Algebra/Group/Units/Opposite.lean,Mathlib/Algebra/Notation/Pi/Basic.lean,Mathlib/Algebra/Opposites.lean,Mathlib/Algebra/Order/BigOperators/Group/List.lean,Mathlib/Algebra/Order/Group/Abs.lean,Mathlib/Algebra/Order/Group/Basic.lean,Mathlib/Algebra/Order/Group/Cone.lean,Mathlib/Algebra/Order/Group/OrderIso.lean,Mathlib/Algebra/Order/Group/Units.lean,Mathlib/Algebra/Order/Hom/Monoid.lean,Mathlib/Algebra/Order/Monoid/Basic.lean,Mathlib/Algebra/Order/Monoid/Canonical/Defs.lean,Mathlib/Algebra/Order/Monoid/Submonoid.lean,Mathlib/Algebra/Order/Monoid/Unbundled/Basic.lean,Mathlib/Algebra/Order/Monoid/Unbundled/WithTop.lean,Mathlib/Algebra/Order/Monoid/Units.lean,Mathlib/Algebra/Order/Pi.lean,Mathlib/Algebra/Regular/Defs.lean,Mathlib/Analysis/Normed/Group/Basic.lean,Mathlib/CategoryTheory/Monoidal/Discrete.lean,Mathlib/Data/Finset/NoncommProd.lean,Mathlib/Data/Fintype/BigOperators.lean,Mathlib/Data/Set/MulAntidiagonal.lean,Mathlib/Data/Set/SMulAntidiagonal.lean,Mathlib/Data/Vector/Basic.lean,Mathlib/Dynamics/Ergodic/Action/OfMinimal.lean,Mathlib/Dynamics/FixedPoints/Prufer.lean,Mathlib/Geometry/Manifold/Algebra/SmoothFunctions.lean,Mathlib/GroupTheory/Complement.lean,Mathlib/GroupTheory/Congruence/Basic.lean,Mathlib/GroupTheory/Congruence/Defs.lean,Mathlib/GroupTheory/Coprod/Basic.lean,Mathlib/GroupTheory/Coset/Basic.lean,Mathlib/GroupTheory/Divisible.lean,Mathlib/GroupTheory/EckmannHilton.lean,Mathlib/GroupTheory/FreeGroup/Basic.lean,Mathlib/GroupTheory/FreeGroup/Reduce.lean,Mathlib/GroupTheory/GroupAction/Basic.lean,Mathlib/GroupTheory/GroupAction/Blocks.lean,Mathlib/GroupTheory/GroupAction/Defs.lean,Mathlib/GroupTheory/GroupAction/FixedPoints.lean,Mathlib/GroupTheory/GroupAction/Hom.lean,Mathlib/GroupTheory/GroupAction/MultipleTransitivity.lean,Mathlib/GroupTheory/GroupAction/Primitive.lean,Mathlib/GroupTheory/GroupAction/Quotient.lean,Mathlib/GroupTheory/GroupAction/SubMulAction.lean |
141 |
10 |
['eric-wieser', 'github-actions', 'grunweg', 'mathlib4-merge-conflict-bot', 'thorimur'] |
nobody |
29-51718 29 days ago |
30-39090 30 days ago |
0-61617 17 hours |
27953 |
CoolRmal author:CoolRmal |
feat(ProbabilityTheory): Conditional Jensen's Inequality |
This PR adds conditional Jensen's inequality.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-measure-probability
merge-conflict
|
526/14 |
Mathlib.lean,Mathlib/Analysis/NormedSpace/HahnBanach/Separation.lean,Mathlib/MeasureTheory/Function/ConditionalExpectation/Basic.lean,Mathlib/MeasureTheory/Function/ConditionalExpectation/CondJensen.lean,Mathlib/MeasureTheory/MeasurableSpace/Constructions.lean |
5 |
3 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
29-49703 29 days ago |
29-49704 29 days ago |
8-36460 8 days |
27759 |
plp127 author:plp127 |
chore(FreeAbelianGroup): deprecate multiplication |
Deprecate multiplication on `FreeAbelianGroup` in favor of using `MonoidAlgebra`.
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebra
merge-conflict
label:t-algebra$ |
176/86 |
Mathlib/Algebra/Algebra/Hom.lean,Mathlib/Algebra/MonoidAlgebra/MapDomain.lean,Mathlib/GroupTheory/FreeAbelianGroup.lean,Mathlib/RingTheory/FreeCommRing.lean,Mathlib/RingTheory/FreeRing.lean |
5 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
29-6906 29 days ago |
29-6907 29 days ago |
14-59974 14 days |
8102 |
miguelmarco author:miguelmarco |
feat(Tactic): add `unify_denoms` and `collect_signs` tactics |
This PR adds four new tactics:
- `unify_denoms` tries to put expressions with several divisions in a form with only one division. In the case of fields, it works similarly to `field_simp`, but if the hypothesis about denominators being nonzero are not present, it assumes them, and leaves them as new goals to prove. In that sense, it is an "unsafe" tactic (but can be useful nevertheless, for example when you can't find which exact hypothesis is missing). It also works with expressions of naturals and Euclidean domains, assuming the corresponding hypothesis about the denominators dividing the numerators.
- `unify_denoms!` extends `unify_denoms` to work with (in)equalities, assuming also that the denominators, once in normal form, are positive.
- `collect_signs` works similarly with expressions using sums and substractions: it tries to put them in a form of one sum minus other sum. In the case of working with naturals, it assumes that we never substract a bigger number from a smaller one.
Both are implemented essentially as a macro that combines several rewriting rules. Some new lemmas with the corresponding rules are added.
--- |
new-contributor
t-meta
merge-conflict
please-adopt
modifies-tactic-syntax
good first issue
|
407/0 |
Mathlib.lean,Mathlib/Algebra/EuclideanDomain/Basic.lean,Mathlib/Tactic.lean,Mathlib/Tactic/CollectSigns.lean,Mathlib/Tactic/UnifyDenoms.lean,MathlibTest/unify_denoms.lean,scripts/noshake.json |
7 |
55 |
['Paul-Lez', 'YaelDillies', 'github-actions', 'joneugster', 'kbuzzard', 'mathlib4-merge-conflict-bot', 'miguelmarco'] |
nobody |
29-4375 29 days ago |
29-14131 29 days ago |
22-16933 22 days |
14203 |
dagurtomas author:dagurtomas |
feat(Algebra/ModuleCat): descent data |
Co-authored-by: Jack McKoen
Co-authored-by: Christian Merten
Co-authored-by: Joël Riou
Co-authored-by: Adam Topaz
---
- [ ] depends on: #24530
[](https://gitpod.io/from-referrer/)
|
workshop-AIM-AG-2024
t-algebra
t-algebraic-geometry
t-category-theory
merge-conflict
WIP
label:t-algebra$ |
253/15 |
Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/ChangeOfRings.lean,Mathlib/Algebra/Category/ModuleCat/Descent.lean,Mathlib/Algebra/Homology/ShortComplex/ExactFunctor.lean,Mathlib/Algebra/Ring/Equiv.lean,Mathlib/AlgebraicGeometry/Morphisms/RingHomProperties.lean,Mathlib/RingTheory/Flat/FaithfullyFlat/Basic.lean,Mathlib/RingTheory/LocalProperties/Basic.lean,Mathlib/RingTheory/RingHom/FaithfullyFlat.lean,Mathlib/RingTheory/RingHom/Finite.lean,Mathlib/RingTheory/RingHom/Flat.lean,Mathlib/RingTheory/RingHom/Integral.lean,Mathlib/RingTheory/RingHom/Locally.lean,Mathlib/RingTheory/RingHom/Surjective.lean,Mathlib/RingTheory/RingHom/Unramified.lean,Mathlib/RingTheory/RingHomProperties.lean |
16 |
4 |
['dagurtomas', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
28-63876 28 days ago |
28-63878 28 days ago |
0-0 0 seconds |
21776 |
alreadydone author:alreadydone |
Invertible modules |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
label:t-algebra$ |
571/26 |
Mathlib/Algebra/Algebra/Operations.lean,Mathlib/Algebra/Module/Submodule/Equiv.lean,Mathlib/Data/Set/Semiring.lean,Mathlib/RingTheory/FractionalIdeal/Operations.lean,Mathlib/RingTheory/PicardGroup.lean |
5 |
3 |
['alreadydone', 'github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
28-6455 28 days ago |
28-6456 28 days ago |
0-0 0 seconds |
20722 |
ctchou author:ctchou |
feat(Counterexamples): the Vitali set is non-measurable |
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-measure-probability
merge-conflict
please-adopt
awaiting-author
|
258/3 |
Counterexamples.lean,Counterexamples/VitaliSetNotMeasurable.lean,Mathlib/MeasureTheory/Measure/NullMeasurable.lean,docs/1000.yaml |
4 |
76 |
['ctchou', 'github-actions', 'grunweg', 'mathlib4-merge-conflict-bot', 'vihdzp'] |
vihdzp assignee:vihdzp |
27-83201 27 days ago |
28-11689 28 days ago |
0-0 0 seconds |
27446 |
grunweg author:grunweg |
chore: more enorm lemmas |
Nothing to see yet: this is a big mess!
Start unrolling at `eLpNorm_le_eLpNorm_top_mul_eLpNorm_enorm`; that proof could be a good next target.
Need a version of `eLpNorm'_const_smul' which applies to NNReal (or ENNReal, I guess): need to generalise a bunch of lemmas for that.
---
[](https://gitpod.io/from-referrer/)
|
carleson
merge-conflict
WIP
|
107/9 |
Mathlib/MeasureTheory/Function/LpSeminorm/Basic.lean,Mathlib/MeasureTheory/Function/LpSeminorm/CompareExp.lean,Mathlib/MeasureTheory/Integral/IntegrableOn.lean |
3 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-merge-conflict-bot'] |
nobody |
27-74715 27 days ago |
27-74716 27 days ago |
0-172 2 minutes |
14583 |
lecopivo author:lecopivo |
fix: make concrete cycle notation local |
fix: make c[...] notation for concrete cycles local
---
The notation for concrete cycles prevents you using `c[i]` notation for `c : Array _`
This currently does not work
```
import Mathlib
variable (c : Array Nat) (i : Fin c.size)
#check c[i] -- breaks because of notation for concrete cycles
```
This PR just marks it as local to prevent this issue.
[](https://gitpod.io/from-referrer/)
|
merge-conflict
awaiting-author
|
1/1 |
Mathlib/GroupTheory/Perm/Cycle/Concrete.lean |
1 |
3 |
['eric-wieser', 'github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
26-7629 26 days ago |
26-7630 26 days ago |
0-12793 3 hours |
27819 |
BGuillemet author:BGuillemet |
feat(CategoryTheory/Yoneda): add curried version of Yoneda lemma for heterogeneous universes, and other version of homNatIso |
Prove a curried version of `yonedaCompUliftFunctorEquiv`, ie a completely functorial version of the Yoneda lemma with heterogeneous universes. Dually, prove a curried version of `coyonedaCompUliftFunctorEquiv`, ie a completely functorial version of the coYoneda lemma with heterogeneous universes.
In addition, prove a functorial version of `FullyFaithful.natEquiv` using `coyoneda` instead of `yoneda` (previously, the only functorial version of `FullyFaithful.natEquiv` were `homNatIso`, which is written using `yoneda`).
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-category-theory
merge-conflict
awaiting-author
|
162/36 |
Mathlib/CategoryTheory/Yoneda.lean |
1 |
4 |
['BGuillemet', 'github-actions', 'joelriou', 'mathlib4-merge-conflict-bot'] |
nobody |
25-83554 25 days ago |
25-83555 25 days ago |
2-57237 2 days |
19097 |
Vierkantor author:Vierkantor |
chore(Algebra.Polynomial): split `Polynomial/Basic.lean` into smaller files |
This PR splits `Mathlib.Algebra.Polynomial.Basic` into the following files:
* `Polynomial/Defs.lean`: definition and ring structure on `R[X]`
* `Polynomial/Module.lean`: module structure on `R[X]`
* `Polynomial/Monomial.lean`: merged definition of `monomial`, `X`, `C` into the existing file (this is probably the file you want to import from now on)
* `Polynomial/EraseUpdate.lean`: definition of `erase` and `update`
* `Polynomial/Sum.lean`: definition of `sum`
Initially I added the monomial results to a new file, but ended up merging it with `Monomial.lean` since the two of them merge cleanly.
---
- [x] depends on: #28030 (going to resurrect this PR on top of that one later)
- [x] depends on: #19095
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
label:t-algebra$ |
3109/2500 |
Mathlib.lean,Mathlib/Algebra/BigOperators/Finsupp.lean,Mathlib/Algebra/MonoidAlgebra/Basic.lean,Mathlib/Algebra/MonoidAlgebra/Defs.lean,Mathlib/Algebra/MonoidAlgebra/Division.lean,Mathlib/Algebra/MonoidAlgebra/Lift.lean,Mathlib/Algebra/MonoidAlgebra/MapDomain.lean,Mathlib/Algebra/MonoidAlgebra/Module.lean,Mathlib/Algebra/MonoidAlgebra/Opposite.lean,Mathlib/Algebra/MonoidAlgebra/Support.lean,Mathlib/Algebra/Polynomial/Basic.lean,Mathlib/Algebra/Polynomial/Cardinal.lean,Mathlib/Algebra/Polynomial/Coeff.lean,Mathlib/Algebra/Polynomial/Defs.lean,Mathlib/Algebra/Polynomial/Degree/Definitions.lean,Mathlib/Algebra/Polynomial/Degree/TrailingDegree.lean,Mathlib/Algebra/Polynomial/EraseUpdate.lean,Mathlib/Algebra/Polynomial/Eval/Defs.lean,Mathlib/Algebra/Polynomial/Eval/Degree.lean,Mathlib/Algebra/Polynomial/Module.lean,Mathlib/Algebra/Polynomial/Monomial.lean,Mathlib/Algebra/Polynomial/Sum.lean,Mathlib/Data/Finsupp/Basic.lean,Mathlib/Data/Finsupp/Defs.lean,Mathlib/Data/Finsupp/Ext.lean,Mathlib/Data/Finsupp/Fintype.lean,Mathlib/Data/Finsupp/Indicator.lean,Mathlib/Data/Finsupp/Notation.lean,Mathlib/Data/Finsupp/Pointwise.lean,Mathlib/Data/Finsupp/SMulWithZero.lean,Mathlib/Data/Finsupp/Single.lean,Mathlib/Data/List/ToFinsupp.lean,Mathlib/LinearAlgebra/Matrix/Charpoly/Eigs.lean,Mathlib/RingTheory/KrullDimension/Basic.lean,Mathlib/RingTheory/Polynomial/Opposites.lean,Mathlib/RingTheory/PowerSeries/Basic.lean,Mathlib/Tactic/ExtractGoal.lean,MathlibTest/Polynomial.lean,MathlibTest/instance_diamonds.lean,scripts/noshake.json |
40 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
24-83461 24 days ago |
30-76246 30 days ago |
0-0 0 seconds |
28054 |
EtienneC30 author:EtienneC30 |
feat: an abbreviation for sesquilinear forms |
Define `SesquilinForm R M := M →ₗ⋆[R] M →ₗ[R] R`. Prove that a `SesquilinForm R M` is symmetric if and only if the corresponding matrix is Hermitian.
---
- [ ] depends on: #27873
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
label:t-algebra$ |
181/39 |
Counterexamples/QuadraticForm.lean,Mathlib.lean,Mathlib/Algebra/Lie/TraceForm.lean,Mathlib/LinearAlgebra/BilinearForm/Properties.lean,Mathlib/LinearAlgebra/BilinearForm/TensorProduct.lean,Mathlib/LinearAlgebra/QuadraticForm/Basic.lean,Mathlib/LinearAlgebra/QuadraticForm/Dual.lean,Mathlib/LinearAlgebra/RootSystem/Finite/CanonicalBilinear.lean,Mathlib/LinearAlgebra/RootSystem/OfBilinear.lean,Mathlib/LinearAlgebra/RootSystem/RootPositive.lean,Mathlib/LinearAlgebra/SesquilinearForm.lean,Mathlib/LinearAlgebra/SesquilinearForm/Basic.lean |
12 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
24-80789 24 days ago |
24-80790 24 days ago |
0-0 0 seconds |
28162 |
EtienneC30 author:EtienneC30 |
feat: define positive semidefinite sesquilinear maps |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
label:t-algebra$ |
73/39 |
Counterexamples/QuadraticForm.lean,Mathlib/Algebra/Lie/TraceForm.lean,Mathlib/LinearAlgebra/BilinearForm/Properties.lean,Mathlib/LinearAlgebra/BilinearForm/TensorProduct.lean,Mathlib/LinearAlgebra/QuadraticForm/Basic.lean,Mathlib/LinearAlgebra/QuadraticForm/Dual.lean,Mathlib/LinearAlgebra/RootSystem/Finite/CanonicalBilinear.lean,Mathlib/LinearAlgebra/RootSystem/OfBilinear.lean,Mathlib/LinearAlgebra/RootSystem/RootPositive.lean,Mathlib/LinearAlgebra/SesquilinearForm.lean |
10 |
3 |
['github-actions', 'mathlib4-merge-conflict-bot', 'themathqueen'] |
nobody |
24-80665 24 days ago |
24-80666 24 days ago |
0-0 0 seconds |
28622 |
alreadydone author:alreadydone |
chore(Mathlib): replace `=>` by `↦` |
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict |
51792/51792 |
Mathlib/Algebra/AddTorsor/Basic.lean,Mathlib/Algebra/AddTorsor/Defs.lean,Mathlib/Algebra/Algebra/Basic.lean,Mathlib/Algebra/Algebra/Bilinear.lean,Mathlib/Algebra/Algebra/Defs.lean,Mathlib/Algebra/Algebra/Equiv.lean,Mathlib/Algebra/Algebra/Hom.lean,Mathlib/Algebra/Algebra/Hom/Rat.lean,Mathlib/Algebra/Algebra/NonUnitalHom.lean,Mathlib/Algebra/Algebra/NonUnitalSubalgebra.lean,Mathlib/Algebra/Algebra/Operations.lean,Mathlib/Algebra/Algebra/Opposite.lean,Mathlib/Algebra/Algebra/Prod.lean,Mathlib/Algebra/Algebra/Rat.lean,Mathlib/Algebra/Algebra/Spectrum/Basic.lean,Mathlib/Algebra/Algebra/Spectrum/Pi.lean,Mathlib/Algebra/Algebra/Spectrum/Quasispectrum.lean,Mathlib/Algebra/Algebra/Subalgebra/Basic.lean,Mathlib/Algebra/Algebra/Subalgebra/Centralizer.lean,Mathlib/Algebra/Algebra/Subalgebra/Directed.lean,Mathlib/Algebra/Algebra/Subalgebra/IsSimpleOrder.lean,Mathlib/Algebra/Algebra/Subalgebra/Lattice.lean,Mathlib/Algebra/Algebra/Subalgebra/Matrix.lean,Mathlib/Algebra/Algebra/Subalgebra/Operations.lean,Mathlib/Algebra/Algebra/Subalgebra/Pointwise.lean,Mathlib/Algebra/Algebra/Subalgebra/Prod.lean,Mathlib/Algebra/Algebra/Subalgebra/Unitization.lean,Mathlib/Algebra/Algebra/Tower.lean,Mathlib/Algebra/Algebra/TransferInstance.lean,Mathlib/Algebra/Algebra/Unitization.lean,Mathlib/Algebra/Algebra/ZMod.lean,Mathlib/Algebra/AlgebraicCard.lean,Mathlib/Algebra/BigOperators/Associated.lean,Mathlib/Algebra/BigOperators/Expect.lean,Mathlib/Algebra/BigOperators/Fin.lean,Mathlib/Algebra/BigOperators/Finprod.lean,Mathlib/Algebra/BigOperators/Finsupp/Basic.lean,Mathlib/Algebra/BigOperators/Finsupp/Fin.lean,Mathlib/Algebra/BigOperators/Group/Finset/Basic.lean,Mathlib/Algebra/BigOperators/Group/Finset/Defs.lean,Mathlib/Algebra/BigOperators/Group/Finset/Piecewise.lean,Mathlib/Algebra/BigOperators/Group/Finset/Sigma.lean,Mathlib/Algebra/BigOperators/Group/List/Basic.lean,Mathlib/Algebra/BigOperators/Group/List/Defs.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/Finset.lean,Mathlib/Algebra/BigOperators/Intervals.lean,Mathlib/Algebra/BigOperators/Option.lean,Mathlib/Algebra/BigOperators/Pi.lean,Mathlib/Algebra/BigOperators/Ring/Finset.lean,Mathlib/Algebra/BigOperators/Ring/Multiset.lean,Mathlib/Algebra/Category/AlgCat/Basic.lean,Mathlib/Algebra/Category/AlgCat/Limits.lean,Mathlib/Algebra/Category/AlgCat/Monoidal.lean,Mathlib/Algebra/Category/BialgCat/Basic.lean,Mathlib/Algebra/Category/BoolRing.lean,Mathlib/Algebra/Category/CoalgCat/Basic.lean,Mathlib/Algebra/Category/CoalgCat/ComonEquivalence.lean,Mathlib/Algebra/Category/FGModuleCat/Limits.lean,Mathlib/Algebra/Category/Grp/AB.lean,Mathlib/Algebra/Category/Grp/Adjunctions.lean,Mathlib/Algebra/Category/Grp/Basic.lean,Mathlib/Algebra/Category/Grp/Biproducts.lean,Mathlib/Algebra/Category/Grp/CartesianMonoidal.lean,Mathlib/Algebra/Category/Grp/Colimits.lean,Mathlib/Algebra/Category/Grp/EpiMono.lean,Mathlib/Algebra/Category/Grp/FilteredColimits.lean,Mathlib/Algebra/Category/Grp/Images.lean,Mathlib/Algebra/Category/Grp/Kernels.lean,Mathlib/Algebra/Category/Grp/LargeColimits.lean,Mathlib/Algebra/Category/Grp/LeftExactFunctor.lean,Mathlib/Algebra/Category/Grp/Limits.lean,Mathlib/Algebra/Category/Grp/Preadditive.lean,Mathlib/Algebra/Category/Grp/ZModuleEquivalence.lean,Mathlib/Algebra/Category/Grp/Zero.lean,Mathlib/Algebra/Category/GrpWithZero.lean,Mathlib/Algebra/Category/HopfAlgCat/Basic.lean,Mathlib/Algebra/Category/ModuleCat/Adjunctions.lean,Mathlib/Algebra/Category/ModuleCat/Basic.lean,Mathlib/Algebra/Category/ModuleCat/Biproducts.lean,Mathlib/Algebra/Category/ModuleCat/ChangeOfRings.lean,Mathlib/Algebra/Category/ModuleCat/Colimits.lean,Mathlib/Algebra/Category/ModuleCat/EpiMono.lean,Mathlib/Algebra/Category/ModuleCat/FilteredColimits.lean,Mathlib/Algebra/Category/ModuleCat/Images.lean,Mathlib/Algebra/Category/ModuleCat/Injective.lean,Mathlib/Algebra/Category/ModuleCat/Kernels.lean,Mathlib/Algebra/Category/ModuleCat/Limits.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.lean,Mathlib/Algebra/Category/ModuleCat/Presheaf/Abelian.lean,Mathlib/Algebra/Category/ModuleCat/Presheaf/Colimits.lean,Mathlib/Algebra/Category/ModuleCat/Presheaf/Limits.lean,Mathlib/Algebra/Category/ModuleCat/Presheaf/Pushforward.lean,Mathlib/Algebra/Category/ModuleCat/Presheaf/Sheafify.lean,Mathlib/Algebra/Category/ModuleCat/Products.lean |
3838 |
4 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
24-43940 24 days ago |
24-43941 24 days ago |
0-83357 23 hours |
24793 |
tristan-f-r author:tristan-f-r |
feat: trace of unitarily similar matrices |
adds a theorem relating trace to unitarily similar matrices used in the easy direction of specht's theorem
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
awaiting-author
label:t-algebra$ |
7/0 |
Mathlib/LinearAlgebra/UnitaryGroup.lean |
1 |
4 |
['github-actions', 'j-loreaux', 'mathlib4-merge-conflict-bot', 'tristan-f-r'] |
nobody |
24-39579 24 days ago |
24-39580 24 days ago |
1-55872 1 day |
28532 |
alreadydone author:alreadydone |
chore(Algebra/Ring/Defs): add two classes and extend more |
Add the missing `NonAssocComm(Semi)ring` and modify existing classes to `extends` more to remove some manual instances.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
label:t-algebra$ |
89/70 |
Mathlib/Algebra/Colimit/DirectLimit.lean,Mathlib/Algebra/Ring/Defs.lean,Mathlib/Analysis/Normed/Unbundled/SpectralNorm.lean,Mathlib/LinearAlgebra/CliffordAlgebra/Basic.lean,Mathlib/NumberTheory/SelbergSieve.lean,Mathlib/RingTheory/Localization/Integral.lean,Mathlib/RingTheory/PowerSeries/GaussNorm.lean,Mathlib/RingTheory/Valuation/Discrete/Basic.lean,Mathlib/Tactic/Ring/Basic.lean,MathlibTest/TCSynth.lean |
10 |
17 |
['alreadydone', 'eric-wieser', 'github-actions', 'leanprover-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
23-63803 23 days ago |
23-63804 23 days ago |
2-77063 2 days |
28675 |
vihdzp author:vihdzp |
chore: deprecate `bsup`, `lsub`, `blsub` |
This PR formally deprecates `Ordinal.bsup`, `Ordinal.lsub`, and `Ordinal.blsub`. These arose as ways to construct suprema of ordinals, before we realized it was a much better idea to simply work with the `ConditionallyCompleteLinearOrderBot` structure of `Ordinal`. As a consequence, it gets rid of some longstanding non-deprecated material depending on deprecated material.
---
- [x] depends on: #28677
[](https://gitpod.io/from-referrer/)
|
t-set-theory
merge-conflict
|
315/130 |
Mathlib/Order/IsNormal.lean,Mathlib/SetTheory/Cardinal/Regular.lean,Mathlib/SetTheory/Game/Birthday.lean,Mathlib/SetTheory/Ordinal/Family.lean,Mathlib/SetTheory/Ordinal/NaturalOps.lean,Mathlib/SetTheory/Ordinal/Topology.lean |
6 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
23-57751 23 days ago |
23-71424 23 days ago |
0-0 0 seconds |
27872 |
JovanGerb author:JovanGerb |
chore(gcongr): clean up imports |
This PR removes redundant `gcongr` imports. And when we do import `gcongr`, we now also import the core `@[gcongr]` tags, and also `grw`.
---
[](https://gitpod.io/from-referrer/)
|
large-import
merge-conflict
delegated
|
7/23 |
Archive/Imo/Imo2019Q4.lean,Mathlib/Algebra/ContinuedFractions/Computation/ApproximationCorollaries.lean,Mathlib/Algebra/ContinuedFractions/Computation/Approximations.lean,Mathlib/Algebra/MvPolynomial/SchwartzZippel.lean,Mathlib/Algebra/Order/BigOperators/Expect.lean,Mathlib/Algebra/Order/CauSeq/Basic.lean,Mathlib/Algebra/Order/Chebyshev.lean,Mathlib/Analysis/Convex/Segment.lean,Mathlib/Analysis/Convex/Star.lean,Mathlib/Combinatorics/Additive/PluenneckeRuzsa.lean,Mathlib/Combinatorics/Enumerative/Catalan.lean,Mathlib/Combinatorics/SetFamily/FourFunctions.lean,Mathlib/Combinatorics/SimpleGraph/Density.lean,Mathlib/Combinatorics/SimpleGraph/Triangle/Basic.lean,Mathlib/Data/Nat/Basic.lean,Mathlib/NumberTheory/FLT/Polynomial.lean,Mathlib/NumberTheory/FermatPsp.lean,Mathlib/Order/Basic.lean,Mathlib/Order/Filter/AtTopBot/Archimedean.lean,Mathlib/Tactic/GCongr/CoreAttrs.lean,Mathlib/Topology/EMetricSpace/Paracompact.lean |
21 |
11 |
['JovanGerb', 'bryangingechen', 'github-actions', 'grunweg', 'mathlib-bors', 'mathlib4-merge-conflict-bot'] |
nobody |
23-20121 23 days ago |
23-20121 23 days ago |
4-34325 4 days |
28626 |
alreadydone author:alreadydone |
chore(Archive, Counterexamples): replace => by ↦ |
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict |
288/288 |
Archive/Arithcc.lean,Archive/Examples/IfNormalization/Result.lean,Archive/Examples/IfNormalization/WithoutAesop.lean,Archive/Examples/PropEncodable.lean,Archive/Imo/Imo1959Q1.lean,Archive/Imo/Imo1960Q1.lean,Archive/Imo/Imo1962Q4.lean,Archive/Imo/Imo1972Q5.lean,Archive/Imo/Imo1977Q6.lean,Archive/Imo/Imo1981Q3.lean,Archive/Imo/Imo1987Q1.lean,Archive/Imo/Imo1988Q6.lean,Archive/Imo/Imo1994Q1.lean,Archive/Imo/Imo1998Q2.lean,Archive/Imo/Imo2001Q2.lean,Archive/Imo/Imo2006Q3.lean,Archive/Imo/Imo2006Q5.lean,Archive/Imo/Imo2008Q2.lean,Archive/Imo/Imo2008Q4.lean,Archive/Imo/Imo2011Q3.lean,Archive/Imo/Imo2013Q1.lean,Archive/Imo/Imo2019Q1.lean,Archive/Imo/Imo2024Q5.lean,Archive/MiuLanguage/Basic.lean,Archive/MiuLanguage/DecisionSuf.lean,Archive/OxfordInvariants/Summer2021/Week3P1.lean,Archive/Sensitivity.lean,Archive/Wiedijk100Theorems/AbelRuffini.lean,Archive/Wiedijk100Theorems/AreaOfACircle.lean,Archive/Wiedijk100Theorems/AscendingDescendingSequences.lean,Archive/Wiedijk100Theorems/BallotProblem.lean,Archive/Wiedijk100Theorems/BirthdayProblem.lean,Archive/Wiedijk100Theorems/BuffonsNeedle.lean,Archive/Wiedijk100Theorems/CubingACube.lean,Archive/Wiedijk100Theorems/FriendshipGraphs.lean,Archive/Wiedijk100Theorems/Konigsberg.lean,Archive/Wiedijk100Theorems/Partition.lean,Archive/Wiedijk100Theorems/SumOfPrimeReciprocalsDiverges.lean,Archive/ZagierTwoSquares.lean,Counterexamples/AharoniKorman.lean,Counterexamples/CanonicallyOrderedCommSemiringTwoMul.lean,Counterexamples/CharPZeroNeCharZero.lean,Counterexamples/CliffordAlgebraNotInjective.lean,Counterexamples/DirectSumIsInternal.lean,Counterexamples/GameMultiplication.lean,Counterexamples/Girard.lean,Counterexamples/HomogeneousPrimeNotPrime.lean,Counterexamples/MapFloor.lean,Counterexamples/MonicNonRegular.lean,Counterexamples/Phillips.lean,Counterexamples/Pseudoelement.lean,Counterexamples/QuadraticForm.lean,Counterexamples/SorgenfreyLine.lean,Counterexamples/ZeroDivisorsInAddMonoidAlgebras.lean |
54 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
22-73066 22 days ago |
22-73067 22 days ago |
2-48353 2 days |
26670 |
yu-yama author:yu-yama |
feat(GroupExtension/Abelian): define `conjClassesEquivH1` |
This PR continues the work from #21837.
Original PR: https://github.com/leanprover-community/mathlib4/pull/21837 |
t-algebra
merge-conflict
label:t-algebra$ |
162/5 |
Mathlib.lean,Mathlib/GroupTheory/GroupExtension/Abelian.lean,Mathlib/GroupTheory/GroupExtension/Basic.lean,Mathlib/GroupTheory/GroupExtension/Defs.lean,docs/references.bib |
5 |
3 |
['erdOne', 'github-actions', 'mathlib4-merge-conflict-bot', 'yu-yama'] |
erdOne assignee:erdOne |
22-54143 22 days ago |
22-54144 22 days ago |
49-15167 49 days |
27634 |
agjftucker author:agjftucker |
fix(Analysis/Calculus/Implicit): consistently rename {`map`, `fun`, `function`} to `fun` |
There are several clear naming issues in the file Implicit.lean, such as
```
theorem prod_map_implicitFunction :
∀ᶠ p : F × G in 𝓝 (φ.prodFun φ.pt), φ.prodFun (φ.implicitFunction p.1 p.2) = p :=
```
where `prod_map` and `prodFun` both refer to the same thing. In this PR I have done my best to resolve these as consistently as possible by renaming everything `map`, also everything `function`, to `fun`. This has the added benefit of making some long names a little shorter.
In passing I rewrapped some comments and replaced `haveI` with `have` where it had been used like `haveI` in Lean 3.
Moves:
- ImplicitFunctionData -> ImplicitFunData
- ImplicitFunctionData.implicitFunction -> ImplicitFunData.implicitFun
- ImplicitFunctionData.prod_map_implicitFunction -> ImplicitFunData.prodFun_implicitFun
- ImplicitFunctionData.left_map_implicitFunction -> ImplicitFunData.leftFun_implicitFun
- ImplicitFunctionData.right_map_implicitFunction -> ImplicitFunData.rightFun_implicitFun
- ImplicitFunctionData.implicitFunction_apply_image -> ImplicitFunData.implicitFun_apply_image
- ImplicitFunctionData.implicitFunction_hasStrictFDerivAt -> ImplicitFunData.hasStrictFDerivAt_implicitFun
- HasStrictFDerivAt.implicitFunctionDataOfComplemented -> HasStrictFDerivAt.implicitFunDataOfComplemented
- HasStrictFDerivAt.implicitFunctionOfComplemented -> HasStrictFDerivAt.implicitFunOfComplemented
- HasStrictFDerivAt.map_implicitFunctionOfComplemented_eq -> HasStrictFDerivAt.map_implicitFunOfComplemented_eq
- HasStrictFDerivAt.eq_implicitFunctionOfComplemented -> HasStrictFDerivAt.eq_implicitFunOfComplemented
- HasStrictFDerivAt.implicitFunctionOfComplemented_apply_image -> HasStrictFDerivAt.implicitFunOfComplemented_apply_image
- HasStrictFDerivAt.to_implicitFunctionOfComplemented -> HasStrictFDerivAt.to_implicitFunOfComplemented
- HasStrictFDerivAt.implicitFunction -> HasStrictFDerivAt.implicitFun
- HasStrictFDerivAt.tendsto_implicitFunction -> HasStrictFDerivAt.tendsto_implicitFun
- _root_.Filter.Tendsto.implicitFunction -> _root_.Filter.Tendsto.implicitFun
- HasStrictFDerivAt.map_implicitFunction_eq -> HasStrictFDerivAt.map_implicitFun_eq
- HasStrictFDerivAt.implicitFunction_apply_image -> HasStrictFDerivAt.implicitFun_apply_image
- HasStrictFDerivAt.eq_implicitFunction -> HasStrictFDerivAt.eq_implicitFun
- HasStrictFDerivAt.to_implicitFunction -> HasStrictFDerivAt.to_implicitFun
---
[](https://gitpod.io/from-referrer/)
|
t-analysis
merge-conflict
|
165/121 |
Mathlib/Analysis/Calculus/Implicit.lean,docs/1000.yaml,docs/overview.yaml,docs/undergrad.yaml |
4 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
22-53513 22 days ago |
22-53514 22 days ago |
23-28425 23 days |
7300 |
ah1112 author:ah1112 |
feat: synthetic geometry |
This is adding synthetic geometry using Avigad's axioms and formalizing Euclid Book I, through the Pythagorean theorem.
---
[](https://gitpod.io/from-referrer/)
|
t-euclidean-geometry
merge-conflict
awaiting-author
help-wanted
|
2661/0 |
Mathlib.lean,Mathlib/Geometry/Synthetic/Avigad/Axioms.lean,Mathlib/Geometry/Synthetic/Avigad/EuclidBookI.lean,Mathlib/Geometry/Synthetic/Avigad/Tactics.lean |
4 |
74 |
['ah1112', 'alreadydone', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'plp127', 'tb65536', 'urkud'] |
nobody |
22-31752 22 days ago |
51-66710 1 month ago |
0-0 0 seconds |
23866 |
kim-em author:kim-em |
chore: remove `[AtLeastTwo n]` hypothesis from the `NatCast` to `OfNat` instance |
This PR observes that we can change
```
instance (priority := 100) instOfNatAtLeastTwo {n : ℕ} [NatCast R] [Nat.AtLeastTwo n] : OfNat R n
```
to
```
instance (priority := 100) instOfNatAtLeastTwo {n : ℕ} [NatCast R] : OfNat R n
```
with minimal fall-out.
A follow-up PR #23867 then observes that we can remove nearly all the `[Nat.AtLeastTwo n]` hypotheses in Mathlib.
This is slightly dangerous -- it does make it more likely that we'll generate non-defeq instances, but it appears to happen very rarely.
However, it will make life slightly easier for something Leo and I are trying to do with `grind` and Grobner bases (we'd like to be able to assume types we consume have `[∀ n, OfNat α n]`, which is possible with this change, but not without...).
Zulip thread: [#PR reviews > #23866 and #23867, removing most `[Nat.AtLeastTwo n]` @ 💬](https://leanprover.zulipchat.com/#narrow/channel/144837-PR-reviews/topic/.2323866.20and.20.2323867.2C.20removing.20most.20.60.5BNat.2EAtLeastTwo.20n.5D.60/near/511157297) |
awaiting-zulip
merge-conflict
|
21/26 |
Mathlib/AlgebraicTopology/FundamentalGroupoid/Basic.lean,Mathlib/Data/Nat/Cast/Defs.lean,Mathlib/Data/Nat/Cast/Order/Basic.lean |
3 |
4 |
['eric-wieser', 'github-actions', 'mathlib4-merge-conflict-bot', 'urkud'] |
nobody |
22-10912 22 days ago |
22-10913 22 days ago |
0-23929 6 hours |
13795 |
astrainfinita author:astrainfinita |
perf(Algebra/{Group, GroupWithZero, Ring}/InjSurj): reduce everything |
---
- [ ] depends on: #15192
- [ ] depends on: #15476
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
label:t-algebra$ |
340/194 |
Mathlib/Algebra/Equiv/TransferInstance.lean,Mathlib/Algebra/Group/InjSurj.lean,Mathlib/Algebra/GroupWithZero/Action/Defs.lean,Mathlib/Algebra/GroupWithZero/Action/End.lean,Mathlib/Algebra/GroupWithZero/InjSurj.lean,Mathlib/Algebra/Module/Defs.lean,Mathlib/Algebra/Module/RingHom.lean,Mathlib/Algebra/Ring/InjSurj.lean,scripts/noshake.json |
9 |
37 |
['MichaelStollBayreuth', 'astrainfinita', 'eric-wieser', 'github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mattrobball'] |
nobody |
21-79137 21 days ago |
151-7742 4 months ago |
52-31623 52 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
t-data
merge-conflict
|
125/17 |
Mathlib/Data/Vector/Basic.lean,Mathlib/Data/Vector/Defs.lean,Mathlib/Logic/Equiv/Array.lean |
3 |
4 |
['github-actions', 'linesthatinterlace', 'mathlib4-merge-conflict-bot', 'robin-carlier'] |
nobody |
21-67797 21 days ago |
21-67798 21 days ago |
66-24122 66 days |
27465 |
erdOne author:erdOne |
feat: the definition of nonarchimedean local fields |
---
- [x] depends on: #27430
- [x] depends on: #27412
- [x] depends on: #27213
[](https://gitpod.io/from-referrer/)
|
t-number-theory
merge-conflict
|
229/21 |
Mathlib.lean,Mathlib/NumberTheory/LocalField/Basic.lean,Mathlib/RingTheory/Valuation/RankOne.lean,Mathlib/RingTheory/Valuation/ValuativeRel.lean,Mathlib/Topology/Algebra/Valued/ValuativeRel.lean |
5 |
20 |
['erdOne', 'github-actions', 'kckennylau', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'pechersky'] |
nobody |
21-61909 21 days ago |
29-7376 29 days ago |
0-4122 1 hour |
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
merge-conflict
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 |
24 |
['dagurtomas', 'eric-wieser', 'github-actions', 'lecopivo', 'mathlib4-merge-conflict-bot'] |
dagurtomas assignee:dagurtomas |
21-58138 21 days ago |
21-58139 21 days ago |
85-19916 85 days |
25775 |
emilyriehl author:emilyriehl |
feat(AlgebraicTopology/SimplicialSet/NerveAdjunction): to Strict Segal 2 |
Under a suitable hypothesis, a map of 2-truncated simplicial sets can be generated from a refl prefunctor between the underlying reflexive quivers --- provided the codomain is `StrictSegal`. This abstracts a previously formalized result that requires the codomain to be the 2-truncated nerve of a category.
Co-authored-by: Aaron Liu
---
The current draft displays the old code for comparison with new versions labeled ALT. After initial review this will be cut.
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #23848.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/23848* |
t-algebraic-topology
infinity-cosmos
t-category-theory
merge-conflict
awaiting-author
|
457/206 |
Mathlib/AlgebraicTopology/SimplexCategory/Basic.lean,Mathlib/AlgebraicTopology/SimplexCategory/Defs.lean,Mathlib/AlgebraicTopology/SimplicialSet/HomotopyCat.lean,Mathlib/AlgebraicTopology/SimplicialSet/NerveAdjunction.lean,Mathlib/AlgebraicTopology/SimplicialSet/StrictSegal.lean,Mathlib/CategoryTheory/ComposableArrows.lean,Mathlib/CategoryTheory/EqToHom.lean |
7 |
38 |
['emilyriehl', 'github-actions', 'joelriou', 'leanprover-community-bot-assistant', 'mathlib4-merge-conflict-bot', 'robin-carlier'] |
robin-carlier assignee:robin-carlier |
21-50765 21 days ago |
21-50766 21 days ago |
17-16247 17 days |
28095 |
Equilibris author:Equilibris |
Univ generic corec |
Draft PR: Adding variable universe corecursor for PFunctor
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
merge-conflict
|
321/70 |
Mathlib/Data/PFunctor/Multivariate/Basic.lean,Mathlib/Data/PFunctor/Multivariate/M.lean,Mathlib/Data/TypeVec.lean |
3 |
7 |
['Equilibris', 'alexkeizer', 'github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
21-40383 21 days ago |
21-40384 21 days ago |
0-0 0 seconds |
28150 |
Equilibris author:Equilibris |
chore: clean up proofs typevec proofs |
While adding variable universe corecs I found a lot of theorems in typevec that could do with a bit of a clean-up
---
[](https://gitpod.io/from-referrer/)
|
t-data
new-contributor
merge-conflict
|
24/26 |
Mathlib/Data/TypeVec.lean |
1 |
7 |
['Equilibris', 'alexkeizer', 'github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
21-40382 21 days ago |
21-40383 21 days ago |
13-49738 13 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
merge-conflict
|
56/49 |
Mathlib/Tactic/Widget/LibraryRewrite.lean,MathlibTest/LibraryRewrite.lean,MathlibTest/rewrites.lean |
3 |
6 |
['YaelDillies', 'erdOne', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-merge-conflict-bot'] |
alexjbest assignee:alexjbest |
21-24137 21 days ago |
21-24137 21 days ago |
41-80687 41 days |
27868 |
grunweg author:grunweg |
linter indentation playground |
---
Trying out the changes in #27525.
[](https://gitpod.io/from-referrer/)
|
t-linter
merge-conflict
WIP
|
413/0 |
Mathlib/AlgebraicTopology/SimplexCategory/Augmented.lean,Mathlib/AlgebraicTopology/SimplexCategory/GeneratorsRelations/Basic.lean,Mathlib/CategoryTheory/Sites/Coherent/Basic.lean,Mathlib/Data/ENNReal/Basic.lean,Mathlib/Data/EReal/Basic.lean,Mathlib/Data/Nat/Prime/Defs.lean,Mathlib/FieldTheory/RatFunc/Basic.lean,Mathlib/Init.lean,Mathlib/ModelTheory/Algebra/Ring/Basic.lean,Mathlib/ModelTheory/Arithmetic/Presburger/Basic.lean,Mathlib/ModelTheory/Basic.lean,Mathlib/ModelTheory/Graph.lean,Mathlib/ModelTheory/Order.lean,Mathlib/Tactic/Linter/Style.lean,Mathlib/Util/Notation3.lean |
15 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
21-23576 21 days ago |
21-23577 21 days ago |
0-1 1 second |
27403 |
MoritzBeroRoos author:MoritzBeroRoos |
fix: replace probably erroneous usage of ⬝ (with old \cdot) by · (with \centerdot) |
Discussion at [zulip](https://leanprover.zulipchat.com/#narrow/channel/270676-lean4/topic/.5Ccdot.20!.3D.20.5Ccenterdot).
Currently the abbreviations \cdot and \centerdot resolve to different, with the naked eye nearly undistinguishable symbols (despite the c in cdot surely standing for center..).
This pr replaces instances of ⬝ where · was probably meant.
All of the replacement is in comments, except for the file bench_summary.lean which is used for priting the github benchmark results. Since this file is about scientific notation of numbers, sure · was meant to be used, not a rectangle.
[Related](https://github.com/leanprover-community/mathlib4/pull/27399)
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
merge-conflict
|
195/195 |
Mathlib/Algebra/ContinuedFractions/Computation/Approximations.lean,Mathlib/Algebra/DirectSum/Idempotents.lean,Mathlib/Algebra/Lie/Derivation/Basic.lean,Mathlib/Algebra/Module/Equiv/Basic.lean,Mathlib/AlgebraicGeometry/EllipticCurve/DivisionPolynomial/Basic.lean,Mathlib/Analysis/Analytic/Constructions.lean,Mathlib/Analysis/CStarAlgebra/CStarMatrix.lean,Mathlib/Analysis/Calculus/ContDiff/Basic.lean,Mathlib/Analysis/Calculus/ContDiff/Bounds.lean,Mathlib/Analysis/Calculus/FDeriv/Symmetric.lean,Mathlib/Analysis/Fourier/FourierTransformDeriv.lean,Mathlib/Analysis/InnerProductSpace/Dual.lean,Mathlib/Analysis/InnerProductSpace/PiL2.lean,Mathlib/Analysis/Normed/Unbundled/InvariantExtension.lean,Mathlib/Analysis/SpecialFunctions/Complex/CircleAddChar.lean,Mathlib/Combinatorics/Configuration.lean,Mathlib/Combinatorics/SimpleGraph/AdjMatrix.lean,Mathlib/Combinatorics/SimpleGraph/LapMatrix.lean,Mathlib/Data/Matrix/Block.lean,Mathlib/Data/Matrix/ConjTranspose.lean,Mathlib/Data/Matrix/Hadamard.lean,Mathlib/Data/Matrix/Mul.lean,Mathlib/Data/Matrix/Notation.lean,Mathlib/Data/Matrix/Reflection.lean,Mathlib/Data/Matrix/RowCol.lean,Mathlib/Data/Matrix/Vec.lean,Mathlib/FieldTheory/PurelyInseparable/PerfectClosure.lean,Mathlib/Geometry/Manifold/GroupLieAlgebra.lean,Mathlib/GroupTheory/Coxeter/Matrix.lean,Mathlib/LinearAlgebra/CrossProduct.lean,Mathlib/LinearAlgebra/Matrix/BilinearForm.lean,Mathlib/LinearAlgebra/Matrix/DotProduct.lean,Mathlib/LinearAlgebra/Matrix/Nondegenerate.lean,Mathlib/LinearAlgebra/Matrix/Orthogonal.lean,Mathlib/LinearAlgebra/Matrix/PosDef.lean,Mathlib/LinearAlgebra/Matrix/SchurComplement.lean,Mathlib/LinearAlgebra/Matrix/SesquilinearForm.lean,Mathlib/LinearAlgebra/Matrix/Trace.lean,Mathlib/LinearAlgebra/Multilinear/Basic.lean,Mathlib/LinearAlgebra/PerfectPairing/Matrix.lean,Mathlib/LinearAlgebra/Projectivization/Constructions.lean,Mathlib/NumberTheory/NumberField/ProductFormula.lean,Mathlib/NumberTheory/SiegelsLemma.lean,Mathlib/RingTheory/DividedPowers/SubDPIdeal.lean,Mathlib/SetTheory/Ordinal/Veblen.lean,Mathlib/Topology/Algebra/Module/Equiv.lean,Mathlib/Topology/Homeomorph/Lemmas.lean,Mathlib/Topology/Instances/Matrix.lean,scripts/bench_summary.lean |
49 |
5 |
['eric-wieser', 'github-actions', 'grunweg', 'leanprover-community-bot-assistant'] |
nobody |
21-19702 21 days ago |
43-82024 1 month ago |
7-54661 7 days |
28042 |
kckennylau author:kckennylau |
feat(Topology/ValuativeRel): a topological basis indexed by pairs of elements |
---
The pullback PR of #27314 and #27163.
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
merge-conflict
|
140/23 |
Mathlib/RingTheory/Valuation/ValuativeRel.lean,Mathlib/Topology/Algebra/Valued/ValuativeRel.lean |
2 |
3 |
['github-actions', 'grunweg', 'mathlib4-merge-conflict-bot'] |
nobody |
21-19656 21 days ago |
21-19656 21 days ago |
7-4998 7 days |
26015 |
linesthatinterlace author:linesthatinterlace |
feat: Add high-level generalizations from `MonoidHom` lifts |
This PR continues the work from #25296.
Original PR: https://github.com/leanprover-community/mathlib4/pull/25296 |
migrated-from-branch
t-algebra
merge-conflict
label:t-algebra$ |
1251/156 |
Mathlib/Algebra/Category/Ring/FinitePresentation.lean,Mathlib/Algebra/Group/Equiv/Basic.lean,Mathlib/Algebra/Group/Hom/Basic.lean,Mathlib/Algebra/Group/Hom/Defs.lean,Mathlib/Algebra/Group/Subgroup/Basic.lean,Mathlib/Algebra/Polynomial/Div.lean,Mathlib/Algebra/Ring/Equiv.lean,Mathlib/Algebra/Ring/Hom/Basic.lean,Mathlib/Algebra/Ring/Hom/Defs.lean,Mathlib/Data/ZMod/Basic.lean,Mathlib/NumberTheory/DirichletCharacter/Basic.lean,Mathlib/RingTheory/Ideal/Maps.lean |
12 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'linesthatinterlace'] |
nobody |
20-67959 20 days ago |
20-67959 20 days ago |
17-68720 17 days |
27399 |
MoritzBeroRoos author:MoritzBeroRoos |
chore: replace every usage of ⬝ᵥ (with old \cdot) by ·ᵥ (with \centerdot) |
Discussion at [zulip](https://leanprover.zulipchat.com/#narrow/channel/270676-lean4/topic/.5Ccdot.20!.3D.20.5Ccenterdot).
Currently the abbreviations `\cdot` and `\centerdot` resolve to different, with the naked eye nearly undistinguishable symbols (despite the c in cdot surely standing for `center`..):
- `\cdot` gives ⬝ [U+2B1D](https://www.compart.com/en/unicode/U+2B1D) "Black Very Small Square"
- `\centerdot` gives · [U+00B7](https://www.compart.com/en/unicode/U+00B7) "Middle Dot"
Mathlib mostly uses the `\centerdot` variant, except for the dotProduct notation and some probably unsuspecting people wanting \centerdot but getting \cdot in their comments and 6 uses of a notation using the raw `\cdot` without any subscript at `Mathlib\Topology\Homotopy\Product.lean`.
This PR replaces the dot product `⬝ᵥ` with its `\centerdot` counterpart `·ᵥ`. The related PR [here](https://github.com/leanprover/vscode-lean4/pull/639) can then overwrite the `\cdot` abbreviation, to produce the same symbol as the `centerdot` abbreviation does.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
merge-conflict
|
133/133 |
Mathlib/Analysis/CStarAlgebra/CStarMatrix.lean,Mathlib/Analysis/InnerProductSpace/PiL2.lean,Mathlib/Combinatorics/Configuration.lean,Mathlib/Combinatorics/SimpleGraph/AdjMatrix.lean,Mathlib/Combinatorics/SimpleGraph/LapMatrix.lean,Mathlib/Data/Matrix/Block.lean,Mathlib/Data/Matrix/ConjTranspose.lean,Mathlib/Data/Matrix/Hadamard.lean,Mathlib/Data/Matrix/Mul.lean,Mathlib/Data/Matrix/Notation.lean,Mathlib/Data/Matrix/Reflection.lean,Mathlib/Data/Matrix/RowCol.lean,Mathlib/Data/Matrix/Vec.lean,Mathlib/LinearAlgebra/CrossProduct.lean,Mathlib/LinearAlgebra/Matrix/BilinearForm.lean,Mathlib/LinearAlgebra/Matrix/DotProduct.lean,Mathlib/LinearAlgebra/Matrix/Nondegenerate.lean,Mathlib/LinearAlgebra/Matrix/Orthogonal.lean,Mathlib/LinearAlgebra/Matrix/PosDef.lean,Mathlib/LinearAlgebra/Matrix/SchurComplement.lean,Mathlib/LinearAlgebra/Matrix/SesquilinearForm.lean,Mathlib/LinearAlgebra/Matrix/Trace.lean,Mathlib/LinearAlgebra/PerfectPairing/Matrix.lean,Mathlib/LinearAlgebra/Projectivization/Constructions.lean,Mathlib/Topology/Instances/Matrix.lean |
25 |
6 |
['MoritzBeroRoos', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant'] |
nobody |
20-67934 20 days ago |
43-82025 1 month ago |
7-62439 7 days |
27835 |
edegeltje author:edegeltje |
feat(Tactic): ring modulo a given characteristic |
This PR extends the `ring` tactic with a new config argument `char` which will try to reduce all constant terms modulo the given characteristic. This allows `ring` to prove e.g. `(x + y)^3 = x^3 + y^3` in characteristic 3. This is a simpler and faster way to do so than what we had before: `repeat { ring; reduce_mod_char }` becomes `ring (config := { char := 3 })`.
The first step is to split off the required `CharP` definitions, since `Mathlib.Algebra.CharP.Basic` already requires the `ring` tactic.
To perform the reduction modulo the given characteristic, I implemented `reduceCast` which reduces a raw integer, and wrapped it in `reduceResult` that takes a `NormNum.Result` for easy use. We need to pass through quite a few parameters into `reduceResult` so maybe it's worth defining a structure, or reusing `Cache` for this.
Then it's basically a case of replacing every place where `ring` constructs a numeral with a call to `reduceResult`.
Limitations:
* `ring` doesn't attempt to detect the characteristic by itself, you need to pass it in explicitly. Trying to infer a `CharP` instance at each point sounds quite expensive.
* Since the support for `%` in `NormNum` only exists for integers, I implemented the reduction only when a `Ring` instance is available. It is still sound in the semiring case, just not complete.
* We could optimize exponentiation in the specific case where the characteristic `p` is a prime that divides the exponent `n`: `(x + y)^n = x^n + y^n`. I'll leave that to future work.
---
This used to be #10765 by Anne Baanen before the great forkening.
[](https://gitpod.io/from-referrer/)
|
migrated-from-branch
large-import
t-meta
merge-conflict
|
312/133 |
Mathlib/LinearAlgebra/Eigenspace/Basic.lean,Mathlib/RingTheory/MvPolynomial/Basic.lean,Mathlib/Tactic/LinearCombination.lean,Mathlib/Tactic/Module.lean,Mathlib/Tactic/Polyrith.lean,Mathlib/Tactic/Ring/Basic.lean,Mathlib/Tactic/Ring/Compare.lean,Mathlib/Tactic/Ring/RingNF.lean,MathlibTest/ring_compare.lean,MathlibTest/ring_mod_char.lean |
10 |
4 |
['edegeltje', 'github-actions', 'mathlib4-merge-conflict-bot'] |
joneugster assignee:joneugster |
19-71770 19 days ago |
30-39527 30 days ago |
11-83928 11 days |
25889 |
plp127 author:plp127 |
fix(Tactic/Widget/Conv): fix various issues |
Fixes various issues with the `conv?` widget. Closes #25162.
([Zulip thread](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/bug.20in.20.60conv.3F.60))
Specifically, fixes issues with `conv?` where
- when converting a `SubExpr.Pos` to conv directions, it always uses the goal expression as reference, even when working on a hypothesis, this often leads to bad results and makes it unusable on hypotheses
- it refuses to go all the way in to a function (for example in `Nat.succ 0`, you can't access `Nat.succ`)
- it refuses to enter binders where the name of the bound variable contains the character `0` (try it on `∀ (x0 : Nat), x0 = x0`)
- it panics if it can't find a binder name instead of just coming up with one itself, this also means usually you can't enter either side of a non-dependent arrow since those usually don't have binder names (try it on `False → False`)
- you can't enter the type of a binder, you end up going into the body instead (try it on `fun (x : False) => (x.elim : False → Nat) x.elim`)
- you can't partially enter a function, you end up going to the top argument after instead (for example, in the expression `id (id id) 0`, when you click on `id (id id)`, you end up going to `id id`)
---
[](https://gitpod.io/from-referrer/)
|
t-meta
merge-conflict
|
419/84 |
Mathlib/Tactic/Widget/Conv.lean,MathlibTest/conv?.lean |
2 |
5 |
['bryangingechen', 'github-actions', 'mathlib4-merge-conflict-bot', 'plp127'] |
bryangingechen and kmill assignee:kmill assignee:bryangingechen |
19-56227 19 days ago |
19-56228 19 days ago |
70-58775 70 days |
23621 |
astrainfinita author:astrainfinita |
chore: deprecate `LinearOrderedComm{Monoid, Group}WithZero` |
---
[](https://gitpod.io/from-referrer/)
- [x] depends on: #20676
|
t-order
t-algebra
merge-conflict
label:t-algebra$ |
261/205 |
Archive/Imo/Imo1998Q2.lean,Counterexamples/LinearOrderWithPosMulPosEqZero.lean,Mathlib/Algebra/Order/Field/Canonical.lean,Mathlib/Algebra/Order/Field/Rat.lean,Mathlib/Algebra/Order/Floor/Ring.lean,Mathlib/Algebra/Order/GroupWithZero/Canonical.lean,Mathlib/Algebra/Order/GroupWithZero/Finset.lean,Mathlib/Algebra/Order/Hom/Monoid.lean,Mathlib/Algebra/Order/Nonneg/Field.lean,Mathlib/Algebra/Order/Nonneg/Ring.lean,Mathlib/Algebra/Order/Ring/Nat.lean,Mathlib/Combinatorics/Additive/PluenneckeRuzsa.lean,Mathlib/Combinatorics/SimpleGraph/Triangle/Basic.lean,Mathlib/Data/ENNReal/Basic.lean,Mathlib/Data/NNRat/Lemmas.lean,Mathlib/Data/NNReal/Defs.lean,Mathlib/Data/Rat/Cast/Order.lean,Mathlib/FieldTheory/IntermediateField/Adjoin/Defs.lean,Mathlib/FieldTheory/RatFunc/AsPolynomial.lean,Mathlib/GroupTheory/ArchimedeanDensely.lean,Mathlib/NumberTheory/EllipticDivisibilitySequence.lean,Mathlib/NumberTheory/FunctionField.lean,Mathlib/NumberTheory/Ostrowski.lean,Mathlib/RingTheory/Valuation/Archimedean.lean,Mathlib/RingTheory/Valuation/Basic.lean,Mathlib/RingTheory/Valuation/ExtendToLocalization.lean,Mathlib/RingTheory/Valuation/Integers.lean,Mathlib/RingTheory/Valuation/Integral.lean,Mathlib/RingTheory/Valuation/Minpoly.lean,Mathlib/RingTheory/Valuation/Quotient.lean,Mathlib/RingTheory/Valuation/RankOne.lean,Mathlib/RingTheory/Valuation/ValExtension.lean,Mathlib/RingTheory/Valuation/ValuationRing.lean,Mathlib/RingTheory/Valuation/ValuationSubring.lean,Mathlib/SetTheory/Cardinal/Order.lean,Mathlib/Topology/Algebra/Valued/LocallyCompact.lean,Mathlib/Topology/Algebra/Valued/NormedValued.lean,Mathlib/Topology/Algebra/Valued/ValuationTopology.lean,Mathlib/Topology/Algebra/Valued/ValuedField.lean,Mathlib/Topology/Algebra/Valued/WithVal.lean,Mathlib/Topology/Algebra/WithZeroTopology.lean,Mathlib/Topology/UnitInterval.lean,MathlibTest/instance_diamonds.lean,scripts/noshake.json |
44 |
n/a |
['astrainfinita', 'github-actions', 'grunweg', 'leanprover-bot', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
kbuzzard assignee:kbuzzard |
19-51224 19 days ago |
unknown |
unknown |
21950 |
erdOne author:erdOne |
feat(NumberTheory/Padics): the completion of `ℚ` at a finite place is `ℚ_[p]` |
---
[](https://gitpod.io/from-referrer/)
|
t-number-theory
merge-conflict
|
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 |
32 |
['Ruben-VandeVelde', 'erdOne', 'faenuccio', 'github-actions', 'leanprover-community-bot-assistant', 'pechersky', 'smmercuri', 'xroblot'] |
nobody |
19-24820 19 days ago |
67-72853 2 months ago |
79-1228 79 days |
28863 |
yury-harmonic author:yury-harmonic |
ignore: make CI build oleans |
It looks like CI doesn't build oleans unless I open a PR. Or I can't see this workflow.
---
[](https://gitpod.io/from-referrer/)
|
large-import
merge-conflict
|
1123/100 |
Mathlib.lean,Mathlib/Algebra/Group/Defs.lean,Mathlib/Algebra/Group/Finsupp.lean,Mathlib/Algebra/Group/Hom/Defs.lean,Mathlib/Algebra/Group/Nat/Defs.lean,Mathlib/Algebra/Group/Pi/Lemmas.lean,Mathlib/Algebra/Group/Prod.lean,Mathlib/Algebra/Group/Torsion.lean,Mathlib/Algebra/MvPolynomial/Eval.lean,Mathlib/Algebra/MvPolynomial/Expand.lean,Mathlib/Algebra/Order/Floor/Semiring.lean,Mathlib/Algebra/Order/Group/Basic.lean,Mathlib/Algebra/Order/Positive/Field.lean,Mathlib/Algebra/Order/Positive/Ring.lean,Mathlib/Algebra/Polynomial/Eval/Defs.lean,Mathlib/Algebra/Ring/Periodic.lean,Mathlib/Algebra/Ring/Torsion.lean,Mathlib/AlgebraicTopology/DoldKan/Decomposition.lean,Mathlib/Combinatorics/SimpleGraph/Finite.lean,Mathlib/Data/DFinsupp/NeLocus.lean,Mathlib/Data/Finset/Defs.lean,Mathlib/Data/Finset/Filter.lean,Mathlib/Data/Finset/Option.lean,Mathlib/Data/Finsupp/NeLocus.lean,Mathlib/Data/Multiset/Defs.lean,Mathlib/Data/Multiset/Filter.lean,Mathlib/Data/NNRat/Floor.lean,Mathlib/Data/Nat/Count.lean,Mathlib/Data/Nat/Factorial/Basic.lean,Mathlib/Data/Nat/NthRoot/Defs.lean,Mathlib/Data/Nat/NthRoot/Lemmas.lean,Mathlib/Data/Nat/Totient.lean,Mathlib/Data/PNat/Factors.lean,Mathlib/Data/Rat/Floor.lean,Mathlib/Data/Rat/Lemmas.lean,Mathlib/Data/ZMod/ValMinAbs.lean,Mathlib/Dynamics/PeriodicPts/Defs.lean,Mathlib/GroupTheory/OrderOfElement.lean,Mathlib/LinearAlgebra/LinearIndependent/Basic.lean,Mathlib/LinearAlgebra/Matrix/SemiringInverse.lean,Mathlib/Logic/Function/Defs.lean,Mathlib/NumberTheory/ArithmeticFunction.lean,Mathlib/Order/Partition/Finpartition.lean,Mathlib/RingTheory/Polynomial/Cyclotomic/Basic.lean,Mathlib/RingTheory/Polynomial/Cyclotomic/Expand.lean,Mathlib/Tactic/NormNum/Basic.lean,Mathlib/Tactic/Positivity/Basic.lean,MathlibTest/norm_num_ext.lean,MathlibTest/positivity.lean |
49 |
3 |
['github-actions', 'grunweg', 'mathlib4-merge-conflict-bot'] |
nobody |
19-4657 19 days ago |
19-4658 19 days ago |
0-0 0 seconds |
28933 |
artie2000 author:artie2000 |
WIP chore(Data): correct definition for `single_apply` |
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict |
101/98 |
Counterexamples/DirectSumIsInternal.lean,Counterexamples/ZeroDivisorsInAddMonoidAlgebras.lean,Mathlib/Algebra/DirectSum/Basic.lean,Mathlib/Algebra/Group/Finsupp.lean,Mathlib/Algebra/MonoidAlgebra/Defs.lean,Mathlib/Algebra/Polynomial/Basic.lean,Mathlib/Analysis/InnerProductSpace/Projection/FiniteDimensional.lean,Mathlib/Combinatorics/Nullstellensatz.lean,Mathlib/Data/DFinsupp/Defs.lean,Mathlib/Data/DFinsupp/Order.lean,Mathlib/Data/DFinsupp/Sigma.lean,Mathlib/Data/Finsupp/Basic.lean,Mathlib/Data/Finsupp/Lex.lean,Mathlib/Data/Finsupp/Order.lean,Mathlib/Data/Finsupp/SMul.lean,Mathlib/Data/Finsupp/Single.lean,Mathlib/Data/Finsupp/ToDFinsupp.lean,Mathlib/LinearAlgebra/Basis/Basic.lean,Mathlib/LinearAlgebra/Basis/Defs.lean,Mathlib/LinearAlgebra/Basis/Prod.lean,Mathlib/LinearAlgebra/DFinsupp.lean,Mathlib/LinearAlgebra/Finsupp/Defs.lean,Mathlib/LinearAlgebra/Finsupp/LinearCombination.lean,Mathlib/LinearAlgebra/Finsupp/Supported.lean,Mathlib/LinearAlgebra/FreeModule/Basic.lean,Mathlib/LinearAlgebra/FreeModule/Finite/CardQuotient.lean,Mathlib/LinearAlgebra/LinearIndependent/Defs.lean,Mathlib/LinearAlgebra/Matrix/ToLin.lean,Mathlib/LinearAlgebra/Multilinear/DFinsupp.lean,Mathlib/LinearAlgebra/StdBasis.lean,Mathlib/RingTheory/MvPolynomial/Groebner.lean |
31 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
17-39728 17 days ago |
17-39729 17 days ago |
0-75271 20 hours |
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-ring-theory
merge-conflict
|
217/157 |
Mathlib/Algebra/Algebra/Operations.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Affine/Point.lean,Mathlib/NumberTheory/RamificationInertia/Basic.lean,Mathlib/RingTheory/Extension/Basic.lean,Mathlib/RingTheory/Finiteness/Basic.lean,Mathlib/RingTheory/Finiteness/Ideal.lean,Mathlib/RingTheory/HopkinsLevitzki.lean,Mathlib/RingTheory/Ideal/Maps.lean,Mathlib/RingTheory/Ideal/Operations.lean |
9 |
9 |
['alreadydone', 'github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
eric-wieser assignee:eric-wieser |
17-31345 17 days ago |
17-31345 17 days ago |
174-59519 174 days |
27437 |
kckennylau author:kckennylau |
feat(RingTheory/Valuation): some lemmas about comparing with 1 and 0 and with each other |
*From the 2025 Local Class Field Theory Workshop.*
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
merge-conflict
WIP
|
109/22 |
Mathlib/NumberTheory/Padics/ValuativeRel.lean,Mathlib/RingTheory/Valuation/Basic.lean,Mathlib/RingTheory/Valuation/Extension.lean,Mathlib/RingTheory/Valuation/ValuativeRel.lean |
4 |
20 |
['erdOne', 'github-actions', 'kckennylau', 'mathlib4-merge-conflict-bot', 'matthewjasper', 'pechersky'] |
nobody |
16-70515 16 days ago |
16-70516 16 days ago |
14-30610 14 days |
28644 |
kckennylau author:kckennylau |
don't mind me, i just want cache |
---
[](https://gitpod.io/from-referrer/)
|
will-close-soon
merge-conflict
WIP
|
214/24 |
Mathlib.lean,Mathlib/NumberTheory/LocalField/Basic.lean,Mathlib/RingTheory/Valuation/RankOne.lean,Mathlib/RingTheory/Valuation/ValuativeRel.lean,Mathlib/Topology/Algebra/Valued/ValuativeRel.lean |
5 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
16-66747 16 days ago |
16-66747 16 days ago |
0-13 13 seconds |
28708 |
sjh227 author:sjh227 |
feat (Data) : edit DoublyStochastic, add Stochastic to matrix |
edit DoublyStochastic add Stochastic
---
Add the file Stochastic to matrix. Edit DoublyStochastic so that it depends on Stochastic along with a new lemma
|
t-data
new-contributor
merge-conflict
|
249/1 |
Mathlib.lean,Mathlib/Data/Matrix/DoublyStochastic.lean,Mathlib/Data/Matrix/Stochastic.lean |
3 |
26 |
['github-actions', 'j-loreaux', 'mathlib4-merge-conflict-bot', 'sjh227'] |
nobody |
16-58646 16 days ago |
16-58646 16 days ago |
0-78027 21 hours |
27508 |
chrisflav author:chrisflav |
feat(RingTheory): height under ring homomorphism |
We show that if `P` lies over `p`, the height of `P` is bounded by the height of `p` plus the height of the image of `P` in `S ⧸ p S`.
In a follow-up PR, we show that equality holds if `S` satisfies going-down as an `R`-algebra.
Co-authored by: Sihan Su
Co-authored by: Yi Song
---
- [ ] depends on: #28520
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
large-import
merge-conflict
|
118/1 |
Mathlib/Data/Set/Finite/Basic.lean,Mathlib/Data/Set/Function.lean,Mathlib/Logic/Function/Basic.lean,Mathlib/RingTheory/Ideal/KrullsHeightTheorem.lean,Mathlib/RingTheory/Ideal/MinimalPrime/Basic.lean,Mathlib/RingTheory/Ideal/Over.lean,Mathlib/RingTheory/Ideal/Quotient/Operations.lean |
7 |
13 |
['YaelDillies', 'chrisflav', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
16-56220 16 days ago |
16-56221 16 days ago |
1-25924 1 day |
6042 |
MohanadAhmed author:MohanadAhmed |
feat(LinearAlgebra/Matrix/SVD): Singular Value Decomposition of R or C Matrices |
This file provides proves the SVD theorem which decomposes a real/complex matrix into left eigenvectors, singular values block diagonal matrix and right eigenvectors.
Any matrix A (M × N) with rank r = A.rank and with elements in ℝ or ℂ fields can be decompsed into the product of three matrices:
$$A = USV$$
* The three matrices are defined as
- $U$: an M × M matrix containing the left eigenvectors of the matrix
- $S$: an M × N matrix with an r × r block in the upper left corner with nonzero singular values
- $V$: an N × N matrix containing the right eigenvectors of the matrix
Note that
* $S$ is a block matrix $S = [S₁₁, S₁₂; S₂₁, S₂₂]$ with
- $S₁₁$: a diagonal r × r matrix and
- $S₁₂$ : r × (N - r) zero matrix, S₂₁ : (M - r) × r zero matrix and
- $S₂₂$: (M - r) × (N - r) zero matrix
* $U$ is a block column matrix U = [U₁ U₂] with
- $U₁$ : a M × r containing left eigenvectors with nonzero singular values.
- $U₂$ : a M × (M - r) containing left eigenvectors with zero singular values.
* $V$ is a block column matrix V = [V₁ V₂] with
- $V₁$ : a N × r containing right eigenvectors with nonzero singular values.
- $V₂$ : a M × (M - r) containing right eigenvectors with zero singular values.
Since in mathlib the eigenvalues of hermitian matrices are defined in an "arbitrary" undetermined order, we begin by partition the singular values into zero and non-zero values. We partition the corresponding eigenvectors from AᴴA and AAᴴ using similar rearrangements. These are included in `SVD.svdReindex`. The basic API for Column and Row partitioned matrices is from `ColumnRowPartitioned`.
We then proceed to transfer some of the lemmas we need about eigenvector matrices (for example that they are unitary: i.e. inverse is conjugate transpose.). Note that since invertibility in mathlib is defined for square matrices while our matrices are partitioned i.e. N × (N₁ ⊕ N₂) and N ≃ (N ⊕ N₂), Lean cannot apply the Invertible definition. We workaround this were necessary.
Lemma `reduced_spectral_theorem` (`reduced_spectral_theorem'`) shows that AᴴA and AAᴴ, can be reduced to products containing only the non-zero singular eigenvectors. This is later used in proving the main SVD theroem. A few lemmas are provided about the invertibility of the non-zero singular values matrix: `svdσ_inv`, `σ_inv_μ_σ_inv_eq_one`, `IsUnit_det_svdσ`, `IsUnit_det_svdσ_mapK` and `svdσ_inv_mapK`.
To make relating left eigenvectors to right eigenvectors easier we define U₁ = AV₁σ⁻¹ while U₂ is obtained from the eigenvectors of (AAᴴ). This avoid a lengthy reindexing operation with many proofs. The vectors in U₂ have no such issue since they are multiplied by zero singular values anyway.
Co-authored-by: Mohanad Ahmed
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
please-adopt
WIP
label:t-algebra$ |
588/0 |
Mathlib.lean,Mathlib/LinearAlgebra/Matrix/SVD/Defs.lean,Mathlib/LinearAlgebra/Matrix/SVD/Reindex.lean |
3 |
115 |
['MohanadAhmed', 'Vierkantor', 'alexjbest', 'eric-wieser', 'j-loreaux', 'jcommelin', 'mathlib4-merge-conflict-bot', 'sgouezel'] |
nobody |
16-41655 16 days ago |
16-41656 16 days ago |
181-72917 181 days |
28826 |
alreadydone author:alreadydone |
feat(Category): add `SemimoduleCat` |
+ introduce Presemiadditive categories, which generalizes Preadditive categories: the Hom sets are commutative monoids rather than groups, and `comp_zero` and `zero_comp` is no longer automatic. The new file Preadditive/Semi.lean is adapted from Preadditive/Basic.lean, though many contents can't be generalized.
+ generalize Functor.Additive and Functor.Linear to take Presemiadditive categories instead. The former needs a `map_zero` field since it's not automatic for Presemiadditive categories.
+ introduce SemimoduleCat, the category of semimodules (mathlib's Module) over a Semiring. The new file ModuleCat/Semi.lean is copied from ModuleCat/Basic.lean.
TODOs: additive/linear equivalence between SemimoduleCat and ModuleCat and use it to transfer results; monoidal structure on SemimoduleCat; change `CommRing.Pic` to use SemimoduleCat.
---
[](https://gitpod.io/from-referrer/)
|
t-category-theory
awaiting-CI
merge-conflict
|
978/123 |
Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Semi.lean,Mathlib/Algebra/Category/MonCat/Presemiadditive.lean,Mathlib/CategoryTheory/Linear/Basic.lean,Mathlib/CategoryTheory/Preadditive/AdditiveFunctor.lean,Mathlib/CategoryTheory/Preadditive/Basic.lean,Mathlib/CategoryTheory/Preadditive/Biproducts.lean,Mathlib/CategoryTheory/Preadditive/FunctorCategory.lean,Mathlib/CategoryTheory/Preadditive/Semi.lean |
9 |
4 |
['alreadydone', 'github-actions', 'mathlib4-merge-conflict-bot', 'plp127'] |
nobody |
16-36294 16 days ago |
16-50533 16 days ago |
0-1 1 second |
27785 |
staroperator author:staroperator |
chore(Algebra/Group/Submonoid): golf `Nat.addSubmonoidClosure_one` using `simp` |
This should improve the proof readability.
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebra
merge-conflict
label:t-algebra$ |
8/15 |
Mathlib/Algebra/Group/Submonoid/Membership.lean,Mathlib/Algebra/Group/Submonoid/Operations.lean,Mathlib/Algebra/Order/Star/Basic.lean |
3 |
9 |
['github-actions', 'joneugster', 'leanprover-bot', 'mathlib4-merge-conflict-bot', 'staroperator'] |
joneugster assignee:joneugster |
16-24997 16 days ago |
16-24998 16 days ago |
26-34065 26 days |
28148 |
kckennylau author:kckennylau |
feat(Matrix): Simproc and Rw-proc for Matrix Transpose |
Co-authored by Aaron Liu.
```lean
example : !![1, 2, 3; 4, 5, 6]ᵀ = !![1, 4; 2, 5; 3, 6] := by
rw [transpose_of% 2 3]
example : !![1, 2, 3; 4, 5, 6]ᵀ = !![1, 4; 2, 5; 3, 6] := by
rw [transpose_of]
example : !![1, 2, 3; 4, 5, 6]ᵀ = !![1, 4; 2, 5; 3, 6] := by
simp only [matrix_transpose]
```
---
[](https://gitpod.io/from-referrer/)
|
t-meta
merge-conflict
|
267/8 |
Mathlib.lean,Mathlib/Data/Matrix/Notation.lean,Mathlib/LinearAlgebra/UnitaryGroup.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Simproc/Matrix.lean,MathlibTest/Simproc/Matrix.lean,MathlibTest/matrix.lean,scripts/noshake.json |
8 |
32 |
['eric-wieser', 'github-actions', 'kckennylau', 'mathlib4-merge-conflict-bot', 'plp127'] |
eric-wieser assignee:eric-wieser |
16-24868 16 days ago |
16-24869 16 days ago |
16-54453 16 days |
20850 |
vihdzp author:vihdzp |
chore(Logic/Equiv/Basic): extend `sumCompl` API |
We make a couple of redundant arguments implicit, rename two misnamed theorems, and add two new ones.
---
I'm not sure if the theorems I renamed actually had the correct name; if they did, then [`Equiv.Set.sumCompl_symm_apply_of_mem`](https://leanprover-community.github.io/mathlib4_docs/Mathlib/Logic/Equiv/Set.html#Equiv.Set.sumCompl_symm_apply_of_mem) and [`Equiv.Set.sumCompl_symm_apply_of_not_mem`](https://leanprover-community.github.io/mathlib4_docs/Mathlib/Logic/Equiv/Set.html#Equiv.Set.sumCompl_symm_apply_of_not_mem) should be renamed instead to match.
[](https://gitpod.io/from-referrer/)
|
t-data
t-logic
merge-conflict
awaiting-author
|
21/6 |
Mathlib/Logic/Equiv/Basic.lean,Mathlib/Logic/Equiv/Fintype.lean |
2 |
6 |
['eric-wieser', 'github-actions', 'grunweg', 'kbuzzard', 'vihdzp'] |
nobody |
16-24863 16 days ago |
177-19670 5 months ago |
28-73677 28 days |
25135 |
vasnesterov author:vasnesterov |
WIP/test PR for faster `tauto` |
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-meta
merge-conflict
WIP
|
14/6 |
Mathlib/Geometry/Manifold/IsManifold/InteriorBoundary.lean,Mathlib/Tactic/Tauto.lean,scripts/noshake.json |
3 |
5 |
['github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
15-54794 15 days ago |
15-54794 15 days ago |
0-1 1 second |
26510 |
alreadydone author:alreadydone |
feat(Matroid): exchange lemmas involving closure |
---
for #24350
[](https://gitpod.io/from-referrer/)
|
t-data
t-combinatorics
merge-conflict
|
37/0 |
Mathlib/Data/Matroid/Closure.lean |
1 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
kmill assignee:kmill |
15-47044 15 days ago |
15-47045 15 days ago |
60-26324 60 days |
29002 |
grunweg author:grunweg |
chore: move Data/Real/Irrational to RingTheory |
It certainly has nothing to do with data (structure).
---
I'm less sure where to put it instead.
[zulip discussion](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Cleaning.20up.20.60Data.60/with/536301893) suggested this place; in the future, this could also be split.
[](https://gitpod.io/from-referrer/)
|
file-removed
awaiting-zulip
merge-conflict
|
10/10 |
Counterexamples/IrrationalPowerOfIrrational.lean,Mathlib.lean,Mathlib/Analysis/Real/Pi/Irrational.lean,Mathlib/Data/Real/GoldenRatio.lean,Mathlib/NumberTheory/DiophantineApproximation/Basic.lean,Mathlib/NumberTheory/Rayleigh.lean,Mathlib/NumberTheory/Transcendental/Liouville/Basic.lean,Mathlib/RingTheory/Real/Irrational.lean,Mathlib/Tactic/NormNum/Irrational.lean,Mathlib/Topology/Instances/AddCircle/DenseSubgroup.lean,Mathlib/Topology/Instances/Irrational.lean |
11 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
15-45385 15 days ago |
15-45386 15 days ago |
0-67 1 minute |
26097 |
adomani author:adomani |
dev: the relative linter |
---
[](https://gitpod.io/from-referrer/)
|
t-linter
merge-conflict
awaiting-author
WIP
|
316/0 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter/Local.lean,Mathlib/Util/ParseGit.lean |
4 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
15-23564 15 days ago |
15-23565 15 days ago |
0-0 0 seconds |
29012 |
grunweg author:grunweg |
chore: reduce `Topology` imports in `Data` |
---
- [ ] depends on: #28966
[](https://gitpod.io/from-referrer/)
|
file-removed
merge-conflict
|
25/24 |
Archive/Imo/Imo1959Q2.lean,Archive/Imo/Imo1960Q2.lean,Archive/Imo/Imo2008Q3.lean,Archive/Imo/Imo2008Q4.lean,Archive/Sensitivity.lean,Mathlib.lean,Mathlib/Algebra/Star/CHSH.lean,Mathlib/Analysis/Complex/Norm.lean,Mathlib/Analysis/LocallyConvex/WithSeminorms.lean,Mathlib/Analysis/NormedSpace/HomeomorphBall.lean,Mathlib/Analysis/RCLike/Basic.lean,Mathlib/Analysis/Real/Sqrt.lean,Mathlib/Data/Real/CompleteField.lean,Mathlib/Data/Real/Irrational.lean,Mathlib/Data/Real/StarOrdered.lean,Mathlib/NumberTheory/Zsqrtd/ToReal.lean,Mathlib/Tactic/Linter/DirectoryDependency.lean,Mathlib/Tactic/NormNum/RealSqrt.lean,MathlibTest/positivity.lean |
19 |
4 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
15-18991 15 days ago |
15-18991 15 days ago |
1-17268 1 day |
26337 |
mans0954 author:mans0954 |
feat(Analysis/NormedSpace/MStructure): M-ideals |
This PR continues the work from #14369.
Original PR: https://github.com/leanprover-community/mathlib4/pull/14369 |
large-import
t-analysis
merge-conflict
WIP
|
857/40 |
Mathlib/Algebra/Module/End.lean,Mathlib/Algebra/Module/Hom.lean,Mathlib/Algebra/Module/LinearMap/End.lean,Mathlib/Analysis/Normed/Module/Complemented.lean,Mathlib/Analysis/NormedSpace/MStructure.lean |
5 |
n/a |
['github-actions', 'mans0954', 'mathlib4-merge-conflict-bot'] |
nobody |
14-43402 14 days ago |
unknown |
unknown |
26343 |
mans0954 author:mans0954 |
feat(Analysis/Normed/Module/Complemented): The idempotent associated with a complemented subspace |
Given a complemented subspace `p` of a Banach space `E`, with complement `q`, there exists an idempotent `P` in the ring `E →L[𝕜] E` such that `P` has range `p` and kernel `q`. Similarly `1-P` has range `q` and kernel `p`.
See Rudin, Functional Analysis, Theorem 5.16.
---
This PR continues the work from #20330.
Original PR: https://github.com/leanprover-community/mathlib4/pull/20330
[](https://gitpod.io/from-referrer/) |
large-import
t-analysis
awaiting-CI
merge-conflict
WIP
|
185/3 |
Mathlib/Algebra/Module/End.lean,Mathlib/Algebra/Module/Hom.lean,Mathlib/Algebra/Module/LinearMap/End.lean,Mathlib/Analysis/Normed/Module/Complemented.lean,Mathlib/RingTheory/Idempotents.lean |
5 |
3 |
['github-actions', 'mans0954', 'mathlib4-merge-conflict-bot'] |
nobody |
14-43401 14 days ago |
14-43402 14 days ago |
0-0 0 seconds |
28743 |
vihdzp author:vihdzp |
refactor: `Ordinal.IsNormal` → `Order.IsNormal` |
We deprecate `Ordinal.IsNormal` in favor of the more general `Order.IsNormal`.
---
- [ ] depends on: #28740
[](https://gitpod.io/from-referrer/)
|
merge-conflict |
280/156 |
Mathlib.lean,Mathlib/Order/IsNormal.lean,Mathlib/SetTheory/Cardinal/Aleph.lean,Mathlib/SetTheory/Ordinal/Arithmetic.lean,Mathlib/SetTheory/Ordinal/Enum.lean,Mathlib/SetTheory/Ordinal/Exponential.lean,Mathlib/SetTheory/Ordinal/Family.lean,Mathlib/SetTheory/Ordinal/FixedPoint.lean,Mathlib/SetTheory/Ordinal/Topology.lean,Mathlib/SetTheory/Ordinal/Veblen.lean,Mathlib/Topology/Order/Basic.lean,Mathlib/Topology/Order/IsNormal.lean |
12 |
4 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
13-42920 13 days ago |
13-42922 13 days ago |
0-0 0 seconds |
29020 |
grunweg author:grunweg |
chore: squeeze a few non-terminal simps |
Founds by the flexible linter in #28962.
---
- [ ] depends on : #29027
[](https://gitpod.io/from-referrer/)
|
merge-conflict
awaiting-author
|
91/70 |
Mathlib/Algebra/BigOperators/Fin.lean,Mathlib/Algebra/Field/GeomSum.lean,Mathlib/Analysis/CStarAlgebra/SpecialFunctions/PosPart.lean,Mathlib/Analysis/Calculus/LHopital.lean,Mathlib/Analysis/Complex/ValueDistribution/FirstMainTheorem.lean,Mathlib/Analysis/Fourier/FourierTransformDeriv.lean,Mathlib/Analysis/Meromorphic/NormalForm.lean,Mathlib/Analysis/Meromorphic/TrailingCoefficient.lean,Mathlib/Analysis/NormedSpace/MultipliableUniformlyOn.lean,Mathlib/Analysis/ODE/Gronwall.lean,Mathlib/Analysis/Real/Pi/Irrational.lean,Mathlib/Analysis/SpecialFunctions/BinaryEntropy.lean,Mathlib/Analysis/SpecialFunctions/ContinuousFunctionalCalculus/Rpow/IntegralRepresentation.lean,Mathlib/Analysis/SpecialFunctions/Gaussian/FourierTransform.lean,Mathlib/Analysis/SpecialFunctions/MulExpNegMulSq.lean,Mathlib/Analysis/SpecialFunctions/MulExpNegMulSqIntegral.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Arctan.lean,Mathlib/CategoryTheory/Galois/Basic.lean,Mathlib/CategoryTheory/Monoidal/DayConvolution/Braided.lean,Mathlib/CategoryTheory/SmallObject/Construction.lean,Mathlib/Combinatorics/Additive/VerySmallDoubling.lean,Mathlib/Combinatorics/Enumerative/Composition.lean,Mathlib/Combinatorics/SetFamily/FourFunctions.lean,Mathlib/Combinatorics/SetFamily/KruskalKatona.lean,Mathlib/Combinatorics/SimpleGraph/ConcreteColorings.lean,Mathlib/Combinatorics/SimpleGraph/Connectivity/WalkDecomp.lean,Mathlib/Combinatorics/SimpleGraph/Regularity/Uniform.lean,Mathlib/Data/Nat/Digits/Lemmas.lean,Mathlib/Geometry/Manifold/MFDeriv/Basic.lean,Mathlib/Geometry/Manifold/Riemannian/Basic.lean,Mathlib/GroupTheory/Coxeter/Basic.lean,Mathlib/GroupTheory/GroupAction/MultiplePrimitivity.lean,Mathlib/GroupTheory/GroupAction/MultipleTransitivity.lean,Mathlib/GroupTheory/GroupAction/SubMulAction/OfStabilizer.lean,Mathlib/LinearAlgebra/TensorProduct/Associator.lean,Mathlib/MeasureTheory/Integral/IntervalIntegral/Periodic.lean,Mathlib/NumberTheory/NumberField/InfinitePlace/Basic.lean,Mathlib/NumberTheory/Zsqrtd/Basic.lean,Mathlib/Order/KrullDimension.lean,Mathlib/Order/OrderIsoNat.lean,Mathlib/Probability/ProbabilityMassFunction/Constructions.lean,Mathlib/RingTheory/HahnSeries/Lex.lean,Mathlib/RingTheory/KrullDimension/Module.lean,Mathlib/RingTheory/MvPowerSeries/Substitution.lean,Mathlib/RingTheory/Polynomial/Cyclotomic/Eval.lean,Mathlib/Tactic/NormNum/Irrational.lean,Mathlib/Topology/Algebra/InfiniteSum/UniformOn.lean,Mathlib/Topology/Order.lean,Mathlib/Topology/PartitionOfUnity.lean |
49 |
31 |
['YaelDillies', 'b-mehta', 'github-actions', 'grunweg', 'mathlib4-merge-conflict-bot', 'vlad902'] |
nobody |
12-62940 12 days ago |
12-62940 12 days ago |
0-1958 32 minutes |
28224 |
joelriou author:joelriou |
feat(AlgebraicTopology): the type of non degenerate simplices of a simplicial set |
---
- [x] depends on: #27968
- [ ] depends on: #28034
- [ ] depends on: #26076
[](https://gitpod.io/from-referrer/)
|
t-algebraic-topology
merge-conflict
WIP
|
490/5 |
Mathlib.lean,Mathlib/AlgebraicTopology/SimplexCategory/Basic.lean,Mathlib/AlgebraicTopology/SimplicialSet/Degenerate.lean,Mathlib/AlgebraicTopology/SimplicialSet/NonDegenerateSimplices.lean,Mathlib/AlgebraicTopology/SimplicialSet/Simplices.lean,Mathlib/AlgebraicTopology/SimplicialSet/StdSimplex.lean,Mathlib/CategoryTheory/EpiMono.lean |
7 |
4 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
12-3933 12 days ago |
12-3935 12 days ago |
0-2 2 seconds |
26931 |
javra author:javra |
feat(CategoryTheory/Enriched): `V`-enriched isomorphisms |
Defines isomorphisms in `V`-enriched categories and relate them to ordinary isomorphisms in the case of ordinary enriched categories.
---
[](https://gitpod.io/from-referrer/)
|
infinity-cosmos
t-category-theory
merge-conflict
awaiting-author
|
211/14 |
Mathlib.lean,Mathlib/CategoryTheory/Enriched/Basic.lean,Mathlib/CategoryTheory/Enriched/Iso.lean,Mathlib/CategoryTheory/Enriched/Opposite.lean,Mathlib/CategoryTheory/Enriched/Ordinary/Basic.lean,Mathlib/CategoryTheory/Enriched/Ordinary/Iso.lean |
6 |
21 |
['emilyriehl', 'github-actions', 'javra', 'joelriou', 'mathlib4-merge-conflict-bot', 'mckoen'] |
nobody |
11-86374 11 days ago |
11-86375 11 days ago |
19-77946 19 days |
28052 |
EtienneC30 author:EtienneC30 |
feat: positive semidefinite sesquilinear forms |
Define positive semidefinite sesquilinear forms and prove that a `SesquilinForm R M` is positive semidefinite if and only if the corresponding matrix is positive semidefinite.
---
- [x] depends on: #27873
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
label:t-algebra$ |
263/39 |
Counterexamples/QuadraticForm.lean,Mathlib.lean,Mathlib/Algebra/Lie/TraceForm.lean,Mathlib/LinearAlgebra/BilinearForm/Properties.lean,Mathlib/LinearAlgebra/BilinearForm/TensorProduct.lean,Mathlib/LinearAlgebra/QuadraticForm/Basic.lean,Mathlib/LinearAlgebra/QuadraticForm/Dual.lean,Mathlib/LinearAlgebra/RootSystem/Finite/CanonicalBilinear.lean,Mathlib/LinearAlgebra/RootSystem/OfBilinear.lean,Mathlib/LinearAlgebra/RootSystem/RootPositive.lean,Mathlib/LinearAlgebra/SesquilinearForm.lean,Mathlib/LinearAlgebra/SesquilinearForm/Basic.lean,Mathlib/LinearAlgebra/SesquilinearForm/IsPosSemidef.lean |
13 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
11-77078 11 days ago |
24-80791 24 days ago |
0-0 0 seconds |
26912 |
pechersky author:pechersky |
chore(Algebra/Ring/Subring): simp tag `Subring.smul_def` |
s-multiplying by a subtype is easiest to manipulate when both terms are in the ambient type. Many places that had to use the _def lemma for a rewrite, or to include it in a simp set, no longer have to.
Ported from #25308
---
[](https://gitpod.io/from-referrer/)
I found this being not-simp frustrating when talking about submodules over a valuation subring. |
maintainer-merge
t-algebra
merge-conflict
label:t-algebra$ |
68/67 |
Mathlib/Algebra/Algebra/Subalgebra/Basic.lean,Mathlib/Algebra/Field/Subfield/Basic.lean,Mathlib/Algebra/Group/Subgroup/Actions.lean,Mathlib/Algebra/Group/Submonoid/MulAction.lean,Mathlib/Algebra/Module/LocalizedModule/Basic.lean,Mathlib/Algebra/Module/LocalizedModule/Exact.lean,Mathlib/Algebra/Module/LocalizedModule/IsLocalization.lean,Mathlib/Algebra/Module/LocalizedModule/Submodule.lean,Mathlib/Algebra/Ring/Periodic.lean,Mathlib/Algebra/Ring/Subring/Basic.lean,Mathlib/Algebra/Ring/Subsemiring/Basic.lean,Mathlib/Analysis/CStarAlgebra/Basic.lean,Mathlib/FieldTheory/KummerExtension.lean,Mathlib/GroupTheory/GroupAction/Defs.lean,Mathlib/GroupTheory/GroupAction/MultiplePrimitivity.lean,Mathlib/GroupTheory/GroupAction/MultipleTransitivity.lean,Mathlib/GroupTheory/GroupAction/SubMulAction/OfFixingSubgroup.lean,Mathlib/GroupTheory/GroupAction/SubMulAction/OfStabilizer.lean,Mathlib/LinearAlgebra/RootSystem/Irreducible.lean,Mathlib/LinearAlgebra/RootSystem/RootPositive.lean,Mathlib/LinearAlgebra/RootSystem/WeylGroup.lean,Mathlib/RingTheory/Etale/Kaehler.lean,Mathlib/RingTheory/LocalProperties/Projective.lean,Mathlib/RingTheory/Localization/InvSubmonoid.lean,Mathlib/RingTheory/OreLocalization/Basic.lean |
25 |
19 |
['artie2000', 'eric-wieser', 'github-actions', 'j-loreaux', 'linesthatinterlace', 'mathlib4-merge-conflict-bot', 'pechersky'] |
joelriou assignee:joelriou |
11-76829 11 days ago |
11-76830 11 days ago |
51-74059 51 days |
22782 |
alreadydone author:alreadydone |
feat(Topology): étalé space associated to a predicate on sections |
---
[](https://gitpod.io/from-referrer/)
|
t-topology
merge-conflict
|
886/160 |
Mathlib.lean,Mathlib/AlgebraicGeometry/ProjectiveSpectrum/StructureSheaf.lean,Mathlib/Data/Set/Operations.lean,Mathlib/Geometry/Manifold/Sheaf/Smooth.lean,Mathlib/Logic/Equiv/Basic.lean,Mathlib/Topology/EtaleSpace.lean,Mathlib/Topology/IsLocalHomeomorph.lean,Mathlib/Topology/Sheaves/LocalPredicate.lean,Mathlib/Topology/Sheaves/Sheafify.lean,Mathlib/Topology/Sheaves/Stalks.lean |
10 |
16 |
['AntoineChambert-Loir', 'alreadydone', 'github-actions', 'jcommelin', 'leanprover-community-bot-assistant', 'mathlib4-merge-conflict-bot'] |
PatrickMassot assignee:PatrickMassot |
11-75198 11 days ago |
38-39554 1 month ago |
30-3459 30 days |
27887 |
JovanGerb author:JovanGerb |
feat: `to_dual` attribute |
This PR defines the `to_dual` attribute for translating lemmas to their dual. This is useful in order theory and in category theory. It is built on top of the `to_additive` machinery.
This PR only adds `@[to_dual]` tags in files that directly need to import `ToDual`, namely `Order/Defs/PartialOrder`, `Order/Notation` and `Combinatorics/Quiver/Basic`. Further tagging is left for (many) future PRs.
This PR continues the work from #21719
This PR depends on/supersedes #27894
Related (mathlib3) issues:
- https://github.com/leanprover-community/mathlib3/issues/13461
- https://github.com/leanprover-community/mathlib3/issues/7691
Co-authored-by: @bryangingechen
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-meta
merge-conflict
|
614/291 |
Mathlib.lean,Mathlib/Combinatorics/Quiver/Basic.lean,Mathlib/GroupTheory/Coset/Defs.lean,Mathlib/Order/Basic.lean,Mathlib/Order/Defs/PartialOrder.lean,Mathlib/Order/Notation.lean,Mathlib/Tactic.lean,Mathlib/Tactic/ToAdditive/Frontend.lean,Mathlib/Tactic/ToAdditive/GuessName.lean,Mathlib/Tactic/ToAdditive/ToDual.lean,Mathlib/Tactic/ToDual.lean,MathlibTest/toAdditive.lean,scripts/noshake.json |
13 |
12 |
['JovanGerb', 'bryangingechen', 'github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
11-57750 11 days ago |
11-57751 11 days ago |
17-18867 17 days |
28820 |
yury-harmonic author:yury-harmonic |
feat(PeriodicPts, OrderOfElement): add `nontriviality` lemmas |
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict |
27/22 |
Mathlib/Dynamics/PeriodicPts/Defs.lean,Mathlib/GroupTheory/OrderOfElement.lean,Mathlib/Logic/Function/Defs.lean |
3 |
3 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
11-57382 11 days ago |
11-57383 11 days ago |
8-81045 8 days |
25208 |
erdOne author:erdOne |
feat(LinearAlgebra): `tensor_induction` macro |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
RFC
merge-conflict
WIP
label:t-algebra$ |
87/116 |
Mathlib/Algebra/Category/ModuleCat/ChangeOfRings.lean,Mathlib/Algebra/Central/TensorProduct.lean,Mathlib/LinearAlgebra/DirectSum/Finsupp.lean,Mathlib/LinearAlgebra/TensorProduct/Basic.lean,Mathlib/RingTheory/Flat/Equalizer.lean,Mathlib/RingTheory/TensorProduct/Basic.lean,Mathlib/RingTheory/TensorProduct/Finite.lean,Mathlib/RingTheory/Unramified/Finite.lean |
8 |
8 |
['chrisflav', 'eric-wieser', 'github-actions', 'leanprover-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
11-21341 11 days ago |
11-21341 11 days ago |
0-600 10 minutes |
27817 |
zhuyizheng author:zhuyizheng |
feat: add IMO2025P1 |
Add a solution to IMO2025P1, the original problem statement from https://github.com/jsm28/IMOLean
---
[](https://gitpod.io/from-referrer/)
|
IMO
new-contributor
merge-conflict
|
1443/0 |
Archive.lean,Archive/Imo/Imo2025Q1.lean |
2 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
dwrensha assignee:dwrensha |
10-55205 10 days ago |
10-55206 10 days ago |
32-25131 32 days |
26014 |
CBirkbeck author:CBirkbeck |
feat: define the Eisenstein Series E2 |
This PR continues the work from #24822.
Original PR: https://github.com/leanprover-community/mathlib4/pull/24822
- [ ] depends on : #27606
|
large-import
t-number-theory
merge-conflict
|
981/13 |
Mathlib.lean,Mathlib/Analysis/Asymptotics/Lemmas.lean,Mathlib/Analysis/Complex/Exponential.lean,Mathlib/Analysis/Complex/IntegerCompl.lean,Mathlib/Analysis/Complex/Norm.lean,Mathlib/Analysis/Complex/SummableUniformlyOn.lean,Mathlib/Analysis/Normed/Group/Basic.lean,Mathlib/Analysis/Normed/Module/Basic.lean,Mathlib/Analysis/Normed/Module/FiniteDimension.lean,Mathlib/Analysis/RCLike/Basic.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Cotangent.lean,Mathlib/NumberTheory/ArithmeticFunction.lean,Mathlib/NumberTheory/LSeries/RiemannZeta.lean,Mathlib/NumberTheory/ModularForms/EisensteinSeries/Defs.lean,Mathlib/NumberTheory/ModularForms/EisensteinSeries/E2.lean,Mathlib/NumberTheory/ModularForms/EisensteinSeries/QExpansion.lean,Mathlib/NumberTheory/ModularForms/EisensteinSeries/Summable.lean,Mathlib/NumberTheory/TsumDivsorsAntidiagonal.lean,Mathlib/Topology/Algebra/InfiniteSum/Basic.lean,Mathlib/Topology/Algebra/InfiniteSum/NatInt.lean |
20 |
5 |
['CBirkbeck', 'github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
10-46820 10 days ago |
10-46821 10 days ago |
0-0 0 seconds |
28803 |
astrainfinita author:astrainfinita |
refactor: unbundle algebra from `ENormed*` |
Further speed up the search in the algebraic typeclass hierarchy by avoiding searching for `TopologicalSpace`.
This PR continues the work from #23961.
- Change `ESeminormed(Add)Monoid` and `ENormed(Add)Monoid` so they no longer carry algebraic data.
- Deprecate `ESeminormed(Add)CommMonoid` and `ENormed(Add)CommMonoid` in favor of `ESeminormed(Add)Monoid` and `ENormed(Add)Monoid` with a commutative algebraic typeclass.
|Old|New|
|---|---|
| `[ESeminormed(Add)(Comm)Monoid E]` | `[(Add)(Comm)Monoid E] [ESeminormed(Add)Monoid E]` |
| `[ENormed(Add)(Comm)Monoid]` | `[(Add)(Comm)Monoid E] [ENormed(Add)Monoid]` |
See [Zulip discussion](https://leanprover.zulipchat.com/#narrow/channel/144837-PR-reviews/topic/.2328803.20refactor.3A.20unbundle.20algebra.20from.20.60ENormed*.60/with/536024350)
------------
- [x] depends on: #28813 |
awaiting-zulip
slow-typeclass-synthesis
t-algebra
t-analysis
merge-conflict
label:t-algebra$ |
80/63 |
Mathlib/Analysis/CStarAlgebra/CStarMatrix.lean,Mathlib/Analysis/Normed/Group/Basic.lean,Mathlib/Analysis/Normed/Group/Continuity.lean,Mathlib/Analysis/Normed/Group/InfiniteSum.lean,Mathlib/Analysis/NormedSpace/IndicatorFunction.lean,Mathlib/MeasureTheory/Function/L1Space/AEEqFun.lean,Mathlib/MeasureTheory/Function/L1Space/HasFiniteIntegral.lean,Mathlib/MeasureTheory/Function/L1Space/Integrable.lean,Mathlib/MeasureTheory/Function/LocallyIntegrable.lean,Mathlib/MeasureTheory/Function/LpSeminorm/Basic.lean,Mathlib/MeasureTheory/Function/LpSeminorm/CompareExp.lean,Mathlib/MeasureTheory/Function/LpSeminorm/TriangleInequality.lean,Mathlib/MeasureTheory/Integral/IntegrableOn.lean,Mathlib/MeasureTheory/Integral/IntervalIntegral/Basic.lean |
14 |
28 |
['astrainfinita', 'bryangingechen', 'github-actions', 'grunweg', 'kbuzzard', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'mathlib-bors', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'sgouezel'] |
grunweg assignee:grunweg |
10-38869 10 days ago |
10-38870 10 days ago |
0-20585 5 hours |
23360 |
kim-em author:kim-em |
chore: review of `erw` in `Algebra/Homology/DerivedCategory` |
|
t-algebra
merge-conflict
awaiting-author
label:t-algebra$ |
22/13 |
Mathlib/Algebra/Homology/DerivedCategory/Basic.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/ExtClass.lean,Mathlib/Algebra/Homology/DerivedCategory/SingleTriangle.lean,Mathlib/Algebra/Homology/HomotopyCategory/SingleFunctors.lean,Mathlib/CategoryTheory/Shift/SingleFunctors.lean |
5 |
5 |
['Ruben-VandeVelde', 'github-actions', 'kim-em', 'mathlib4-merge-conflict-bot'] |
nobody |
10-27136 10 days ago |
10-27137 10 days ago |
82-55827 82 days |
26603 |
vihdzp author:vihdzp |
refactor(SetTheory/Ordinal/FixedPoint): redefine `Ordinal.deriv` |
We previously defined the [ordinal derivative](https://en.wikipedia.org/wiki/Normal_function#Properties) of a function as the unique normal function satisfying `deriv f 0 = nfp f 0` and `deriv f (o + 1) = nfp f (deriv f o)` (where `nfp f a` is the next fixed point of `f` that's `≥ a`). The motivation here was to give a "nice" junk value on non-normal functions (the derivative is normal no matter what). However, in practice, this definition makes it unwieldy to prove things, by either requiring a tedious zero/successor/limit argument, or requiring one to rewrite `deriv f = enumOrd (fixedPoints f)`.
We can instead define `deriv f = enumOrd (fixedPoints f)`. At the cost of giving "worse" junk values (which we have no legitimate uses of), we're able to much more easily prove all the expected properties in the standard case where `f` is a normal function.
Finally, we do some drive-by API cleanup.
---
The GitHub diff is a bit messy, I made my best to clean it up.
Moved from #21858.
[](https://gitpod.io/from-referrer/)
|
t-set-theory
merge-conflict
|
173/200 |
Mathlib/SetTheory/Cardinal/Regular.lean,Mathlib/SetTheory/Ordinal/FixedPoint.lean,Mathlib/SetTheory/Ordinal/Veblen.lean |
3 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-merge-conflict-bot'] |
nobody |
10-24557 10 days ago |
10-24558 10 days ago |
12-50686 12 days |
25662 |
erdOne author:erdOne |
chore: redefine `LocalizedModule` |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
label:t-algebra$ |
196/228 |
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 |
14 |
['erdOne', 'eric-wieser', 'github-actions', 'kckennylau', 'leanprover-bot', 'leanprover-community-bot-assistant', 'vihdzp'] |
nobody |
10-21281 10 days ago |
10-21964 10 days ago |
45-34308 45 days |
29345 |
adomani author:adomani |
test: automatically remove deprecations from before 2025-02-31 |
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict |
201/1358 |
Mathlib/Algebra/Category/Grp/Basic.lean,Mathlib/Algebra/Category/MonCat/Basic.lean,Mathlib/Algebra/Order/Field/Canonical.lean,Mathlib/Algebra/Order/Monoid/Canonical/Defs.lean,Mathlib/Algebra/Order/Ring/Canonical.lean,Mathlib/Analysis/InnerProductSpace/Positive.lean,Mathlib/Analysis/InnerProductSpace/Projection/Basic.lean,Mathlib/Combinatorics/Matroid/Circuit.lean,Mathlib/Combinatorics/Matroid/Closure.lean,Mathlib/Combinatorics/Matroid/Minor/Restrict.lean,Mathlib/Computability/Halting.lean,Mathlib/Computability/Partrec.lean,Mathlib/Computability/Primrec.lean,Mathlib/Data/ENNReal/Basic.lean,Mathlib/Data/Fin/Basic.lean,Mathlib/Data/Fin/SuccPred.lean,Mathlib/Data/Finite/Card.lean,Mathlib/Data/Finset/Basic.lean,Mathlib/Data/Fintype/BigOperators.lean,Mathlib/Data/List/Basic.lean,Mathlib/Data/List/Cycle.lean,Mathlib/Data/List/GetD.lean,Mathlib/Data/List/MinMax.lean,Mathlib/Data/List/ModifyLast.lean,Mathlib/Data/List/Nodup.lean,Mathlib/Data/List/NodupEquivFin.lean,Mathlib/Data/List/OfFn.lean,Mathlib/Data/List/ReduceOption.lean,Mathlib/Data/List/Rotate.lean,Mathlib/Data/List/Scan.lean,Mathlib/Data/List/TakeDrop.lean,Mathlib/Data/List/Zip.lean,Mathlib/Data/Matrix/ColumnRowPartitioned.lean,Mathlib/Data/Multiset/Basic.lean,Mathlib/Data/Seq/Defs.lean,Mathlib/Data/Set/Finite/Basic.lean,Mathlib/Data/Set/List.lean,Mathlib/Data/Set/Operations.lean,Mathlib/Data/Set/Prod.lean,Mathlib/Data/Stream/Init.lean,Mathlib/Data/String/Lemmas.lean,Mathlib/Data/Sum/Basic.lean,Mathlib/Geometry/Manifold/ContMDiff/Constructions.lean,Mathlib/Geometry/RingedSpace/Basic.lean,Mathlib/GroupTheory/GroupAction/SubMulAction.lean,Mathlib/GroupTheory/GroupAction/SubMulAction/Pointwise.lean,Mathlib/GroupTheory/Perm/Cycle/Concrete.lean,Mathlib/LinearAlgebra/AffineSpace/AffineSubspace/Basic.lean,Mathlib/LinearAlgebra/Dimension/Constructions.lean,Mathlib/LinearAlgebra/Dimension/RankNullity.lean,Mathlib/LinearAlgebra/LinearIndependent/Basic.lean,Mathlib/LinearAlgebra/LinearIndependent/Defs.lean,Mathlib/LinearAlgebra/LinearIndependent/Lemmas.lean,Mathlib/LinearAlgebra/Matrix/Hermitian.lean,Mathlib/LinearAlgebra/Matrix/PosDef.lean,Mathlib/LinearAlgebra/Matrix/Spectrum.lean,Mathlib/Logic/Equiv/Basic.lean,Mathlib/Logic/Equiv/List.lean,Mathlib/MeasureTheory/Function/ConditionalExpectation/AEMeasurable.lean,Mathlib/MeasureTheory/Function/ConditionalExpectation/Basic.lean,Mathlib/MeasureTheory/Function/ContinuousMapDense.lean,Mathlib/MeasureTheory/Function/L1Space/Integrable.lean,Mathlib/MeasureTheory/Function/L2Space.lean,Mathlib/MeasureTheory/Function/LocallyIntegrable.lean,Mathlib/MeasureTheory/Function/LpOrder.lean,Mathlib/MeasureTheory/Function/LpSeminorm/ChebyshevMarkov.lean,Mathlib/MeasureTheory/Function/LpSeminorm/CompareExp.lean,Mathlib/MeasureTheory/Function/LpSeminorm/Defs.lean,Mathlib/MeasureTheory/Function/LpSeminorm/Trim.lean,Mathlib/MeasureTheory/Function/LpSpace/Basic.lean,Mathlib/MeasureTheory/Function/LpSpace/Complete.lean,Mathlib/MeasureTheory/Function/LpSpace/Indicator.lean,Mathlib/MeasureTheory/Function/StronglyMeasurable/Lp.lean,Mathlib/MeasureTheory/Integral/Bochner/Basic.lean,Mathlib/MeasureTheory/Integral/CircleTransform.lean,Mathlib/MeasureTheory/Integral/IntegrableOn.lean,Mathlib/MeasureTheory/Integral/Lebesgue/Countable.lean,Mathlib/MeasureTheory/Measure/Content.lean,Mathlib/MeasureTheory/Measure/Count.lean,Mathlib/ModelTheory/Basic.lean,Mathlib/ModelTheory/Definability.lean,Mathlib/ModelTheory/ElementarySubstructures.lean,Mathlib/ModelTheory/LanguageMap.lean,Mathlib/ModelTheory/Semantics.lean,Mathlib/ModelTheory/Substructures.lean,Mathlib/ModelTheory/Syntax.lean,Mathlib/NumberTheory/Divisors.lean,Mathlib/NumberTheory/ModularForms/EisensteinSeries/IsBoundedAtImInfty.lean,Mathlib/NumberTheory/NumberField/CanonicalEmbedding/Basic.lean,Mathlib/NumberTheory/NumberField/FinitePlaces.lean,Mathlib/NumberTheory/NumberField/House.lean,Mathlib/Order/Filter/AtTopBot/Monoid.lean,Mathlib/Order/Filter/AtTopBot/Ring.lean,Mathlib/Order/GaloisConnection/Basic.lean,Mathlib/Order/Max.lean,Mathlib/Order/WithBot.lean,Mathlib/Probability/IdentDistrib.lean,Mathlib/Probability/Independence/Integrable.lean,Mathlib/Probability/Kernel/Composition/IntegralCompProd.lean,Mathlib/Probability/Kernel/Invariance.lean |
132 |
0 |
[] |
nobody |
8-72265 8 days ago |
8-72265 8 days ago |
0-49 49 seconds |
29350 |
bryangingechen author:bryangingechen |
test: run script from #27956 on de2995686cbdea3ba481fe421d46bb30b64aae06 |
cf. [#mathlib reviewers > auto-removing oudated deprecations @ 💬](https://leanprover.zulipchat.com/#narrow/channel/345428-mathlib-reviewers/topic/auto-removing.20oudated.20deprecations/near/537719692)
---
#27956
[](https://gitpod.io/from-referrer/)
|
merge-conflict |
0/1124 |
Mathlib/Combinatorics/Matroid/Circuit.lean,Mathlib/Combinatorics/Matroid/Closure.lean,Mathlib/Combinatorics/Matroid/Minor/Restrict.lean,Mathlib/Computability/Halting.lean,Mathlib/Computability/Partrec.lean,Mathlib/Computability/Primrec.lean,Mathlib/Data/ENNReal/Basic.lean,Mathlib/Data/Fin/Basic.lean,Mathlib/Data/Fin/SuccPred.lean,Mathlib/Data/Finite/Card.lean,Mathlib/Data/Finset/Basic.lean,Mathlib/Data/Fintype/BigOperators.lean,Mathlib/Data/List/Basic.lean,Mathlib/Data/List/Cycle.lean,Mathlib/Data/List/GetD.lean,Mathlib/Data/List/MinMax.lean,Mathlib/Data/List/ModifyLast.lean,Mathlib/Data/List/Nodup.lean,Mathlib/Data/List/NodupEquivFin.lean,Mathlib/Data/List/OfFn.lean,Mathlib/Data/List/ReduceOption.lean,Mathlib/Data/List/Rotate.lean,Mathlib/Data/List/Scan.lean,Mathlib/Data/List/TakeDrop.lean,Mathlib/Data/List/Zip.lean,Mathlib/Data/Matrix/ColumnRowPartitioned.lean,Mathlib/Data/Multiset/Basic.lean,Mathlib/Data/Seq/Defs.lean,Mathlib/Data/Set/Finite/Basic.lean,Mathlib/Data/Set/List.lean,Mathlib/Data/Set/Operations.lean,Mathlib/Data/Set/Prod.lean,Mathlib/Data/Stream/Init.lean,Mathlib/Data/String/Lemmas.lean,Mathlib/Data/Sum/Basic.lean,Mathlib/Geometry/Manifold/ContMDiff/Constructions.lean,Mathlib/Geometry/RingedSpace/Basic.lean,Mathlib/GroupTheory/GroupAction/SubMulAction.lean,Mathlib/GroupTheory/Perm/Cycle/Concrete.lean,Mathlib/LinearAlgebra/AffineSpace/AffineSubspace/Basic.lean,Mathlib/LinearAlgebra/Dimension/Constructions.lean,Mathlib/LinearAlgebra/Dimension/RankNullity.lean,Mathlib/LinearAlgebra/LinearIndependent/Basic.lean,Mathlib/LinearAlgebra/LinearIndependent/Defs.lean,Mathlib/LinearAlgebra/LinearIndependent/Lemmas.lean,Mathlib/Logic/Equiv/Basic.lean,Mathlib/Logic/Equiv/List.lean,Mathlib/MeasureTheory/Function/ConditionalExpectation/AEMeasurable.lean,Mathlib/MeasureTheory/Function/ConditionalExpectation/Basic.lean,Mathlib/MeasureTheory/Function/ContinuousMapDense.lean,Mathlib/MeasureTheory/Function/L1Space/Integrable.lean,Mathlib/MeasureTheory/Function/L2Space.lean,Mathlib/MeasureTheory/Function/LocallyIntegrable.lean,Mathlib/MeasureTheory/Function/LpOrder.lean,Mathlib/MeasureTheory/Function/LpSeminorm/ChebyshevMarkov.lean,Mathlib/MeasureTheory/Function/LpSeminorm/CompareExp.lean,Mathlib/MeasureTheory/Function/LpSeminorm/Defs.lean,Mathlib/MeasureTheory/Function/LpSeminorm/Trim.lean,Mathlib/MeasureTheory/Function/LpSpace/Basic.lean,Mathlib/MeasureTheory/Function/LpSpace/Complete.lean,Mathlib/MeasureTheory/Function/LpSpace/Indicator.lean,Mathlib/MeasureTheory/Function/StronglyMeasurable/Lp.lean,Mathlib/MeasureTheory/Integral/Bochner/Basic.lean,Mathlib/MeasureTheory/Integral/CircleTransform.lean,Mathlib/MeasureTheory/Integral/IntegrableOn.lean,Mathlib/MeasureTheory/Integral/Lebesgue/Countable.lean,Mathlib/MeasureTheory/Measure/Content.lean,Mathlib/MeasureTheory/Measure/Count.lean,Mathlib/ModelTheory/Basic.lean,Mathlib/ModelTheory/Definability.lean,Mathlib/ModelTheory/ElementarySubstructures.lean,Mathlib/ModelTheory/LanguageMap.lean,Mathlib/ModelTheory/Semantics.lean,Mathlib/ModelTheory/Substructures.lean,Mathlib/ModelTheory/Syntax.lean,Mathlib/NumberTheory/Divisors.lean,Mathlib/NumberTheory/ModularForms/EisensteinSeries/IsBoundedAtImInfty.lean,Mathlib/NumberTheory/NumberField/CanonicalEmbedding/Basic.lean,Mathlib/NumberTheory/NumberField/FinitePlaces.lean,Mathlib/NumberTheory/NumberField/House.lean,Mathlib/Order/Filter/AtTopBot/Monoid.lean,Mathlib/Order/Filter/AtTopBot/Ring.lean,Mathlib/Order/GaloisConnection/Basic.lean,Mathlib/Order/Max.lean,Mathlib/Order/WithBot.lean,Mathlib/Probability/IdentDistrib.lean,Mathlib/Probability/Independence/Integrable.lean,Mathlib/Probability/Kernel/Composition/IntegralCompProd.lean,Mathlib/Probability/Kernel/Invariance.lean,Mathlib/Probability/Martingale/Convergence.lean,Mathlib/Probability/Moments/ComplexMGF.lean,Mathlib/Probability/Moments/IntegrableExpMul.lean,Mathlib/Probability/Moments/Variance.lean,Mathlib/Probability/Process/Filtration.lean,Mathlib/RingTheory/Algebraic/Integral.lean,Mathlib/RingTheory/AlgebraicIndependent/AlgebraicClosure.lean,Mathlib/RingTheory/AlgebraicIndependent/Basic.lean,Mathlib/RingTheory/Ideal/Maps.lean,Mathlib/RingTheory/NonUnitalSubsemiring/Defs.lean,Mathlib/RingTheory/Spectrum/Prime/Topology.lean |
117 |
0 |
[] |
nobody |
8-61337 8 days ago |
8-61995 8 days ago |
0-0 0 seconds |
26956 |
mariainesdff author:mariainesdff |
feat(RingTheory/DividedPowers/Basic): add divided power structure on pZp |
We construct a divided power structure on the ideal `(p) ⊆ ℤ_[p]`, given by the family of maps `fun n x ↦ x^n / n!`.
Co-authored-by: @AntoineChambert-Loir
---
- [ ] depends on: #22322
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
merge-conflict
|
561/2 |
Mathlib.lean,Mathlib/Data/Nat/Factorial/NatCast.lean,Mathlib/RingTheory/DividedPowers/Padic.lean,Mathlib/RingTheory/DividedPowers/RatAlgebra.lean |
4 |
5 |
['github-actions', 'loefflerd', 'mariainesdff', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
mattrobball assignee:mattrobball |
7-58267 7 days ago |
7-58268 7 days ago |
57-33036 57 days |
27566 |
wwylele author:wwylele |
feat(Data/Real): Archimedean.embedReal is a ring hom when M is an ordered ring |
Also shows that this ends up the same as `LinearOrderedField.inducedOrderRingHom` for fields
---
This is a spin-off from #27268 ~~because I got bored~~ . This is not in a high priority as I don't need it for anything yet, but the last lemma shows that `embedReal` is a generalization of `LinearOrderedField.inducedOrderRingHom` (which is only stated for field, and I didn't find when I was making the group embedding). Perhaps we should refactor `Mathlib/Algebra/Order/CompleteField.lean` with the definition here. Indeed, if we replace every `ℝ` with `(R : Type*)[ConditionallyCompleteLinearOrderedField R]` in `Data/Real/Embedding.lean`, the proof still works. What do you think?
[](https://gitpod.io/from-referrer/)
|
large-import
t-data
merge-conflict
|
220/3 |
Mathlib/Data/Real/Embedding.lean |
1 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
7-17987 7 days ago |
7-17988 7 days ago |
40-32085 40 days |
27918 |
kim-em author:kim-em |
wip: refactor WithBot/WithTop as structures |
For now we are still relying on `WithBot` and `WithTop` being defeq, but there is no impossible obstacle to converting them *both* to the same structure.
This PR begins this effort; the modified files are all compiling, but there are more files that still have problems.
Help on this (either ask to push to my branch, PR to my branch, or just adopt the whole thing!) very much appreciated. |
file-removed
merge-conflict
|
816/330 |
Mathlib.lean,Mathlib/Algebra/Order/AddGroupWithTop.lean,Mathlib/Algebra/Order/GroupWithZero/Canonical.lean,Mathlib/Algebra/Order/Interval/Basic.lean,Mathlib/Algebra/Order/Monoid/ToMulBot.lean,Mathlib/Algebra/Order/Monoid/Unbundled/WithTop.lean,Mathlib/Algebra/Order/Ring/WithTop.lean,Mathlib/CategoryTheory/Preadditive/Injective/Basic.lean,Mathlib/Combinatorics/SimpleGraph/Finite.lean,Mathlib/Data/Countable/Basic.lean,Mathlib/Data/ENNReal/Basic.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/Data/ENat/Defs.lean,Mathlib/Data/Finset/Max.lean,Mathlib/Data/Finset/WithBot.lean,Mathlib/Data/List/MinMax.lean,Mathlib/Data/Nat/PartENat.lean,Mathlib/Data/Ordmap/Invariants.lean,Mathlib/Data/Ordmap/Ordset.lean,Mathlib/Data/Sum/Order.lean,Mathlib/GroupTheory/ArchimedeanDensely.lean,Mathlib/Logic/Embedding/WithBot.lean,Mathlib/Logic/Equiv/WithBot.lean,Mathlib/MeasureTheory/MeasurableSpace/Constructions.lean,Mathlib/Order/Category/BddLat.lean,Mathlib/Order/ConditionallyCompleteLattice/Basic.lean,Mathlib/Order/GaloisConnection/Basic.lean,Mathlib/Order/Hom/WithTopBot.lean,Mathlib/Order/Interval/Basic.lean,Mathlib/Order/Interval/Finset/Defs.lean,Mathlib/Order/Interval/Set/WithBotTop.lean,Mathlib/Order/KrullDimension.lean,Mathlib/Order/Set.lean,Mathlib/Order/SuccPred/Basic.lean,Mathlib/Order/TypeTags.lean,Mathlib/Order/WithBot/Basic.lean,Mathlib/Order/WithBot/NAry.lean,Mathlib/RingTheory/UniqueFactorizationDomain/FactorSet.lean,Mathlib/SetTheory/Cardinal/ENat.lean,Mathlib/Topology/Compactification/OnePoint/Basic.lean,MathlibTest/lift.lean |
41 |
7 |
['eric-wieser', 'github-actions', 'kim-em', 'mathlib4-merge-conflict-bot'] |
nobody |
5-4658 5 days ago |
5-4659 5 days ago |
32-5410 32 days |
27972 |
smmercuri author:smmercuri |
chore: make `Valuation.Completion` a `def` and refactor more of `AdicValuation.lean` |
This PR continues the work from #24590.
Original PR: https://github.com/leanprover-community/mathlib4/pull/24590 |
t-algebra
t-number-theory
merge-conflict
label:t-algebra$ |
174/90 |
Mathlib/NumberTheory/NumberField/FinitePlaces.lean,Mathlib/RingTheory/DedekindDomain/AdicValuation.lean,Mathlib/RingTheory/DedekindDomain/FiniteAdeleRing.lean,Mathlib/RingTheory/LaurentSeries.lean,Mathlib/Topology/Algebra/Valued/WithVal.lean |
5 |
6 |
['github-actions', 'leanprover-bot', 'mathlib4-merge-conflict-bot', 'smmercuri'] |
nobody |
5-4656 5 days ago |
5-4657 5 days ago |
3-74765 3 days |
28151 |
iehality author:iehality |
feat(Computability): r.e. sets are closed under inter/union/projection/composition |
Prove that r.e. sets are closed under intersections, unions, projection and composition.
---
This PR continues the work from #16705.
Original PR: https://github.com/leanprover-community/mathlib4/pull/16705 |
t-computability
merge-conflict
awaiting-author
|
120/0 |
Mathlib/Computability/Halting.lean |
1 |
13 |
['YaelDillies', 'github-actions', 'iehality', 'mathlib4-merge-conflict-bot'] |
YaelDillies assignee:YaelDillies |
5-4532 5 days ago |
5-4533 5 days ago |
9-70671 9 days |
12143 |
adomani author:adomani |
feat: generic linter, absorbing `cdot` linter and `attribute [instance] in` linter |
A "generic" syntax linter that can be configured using a function `Syntax → Array Syntax`.
The expectations is that the function returns sub-syntax extracted from the input that should be flagged by the linter.
This PR provides two examples.
* Flags uses of `cdot` that are not typed as `·`.
* #12137
is a PR that inspired this one.
* Flag uses of `attribute [instance] in` that is not limited to the next declaration
* Inspired by the existing PR by Michael Rothgang
#13190
---
[](https://gitpod.io/from-referrer/)
|
t-linter
merge-conflict
|
210/2 |
Mathlib.lean,Mathlib/Combinatorics/Colex.lean,Mathlib/NumberTheory/LegendreSymbol/AddCharacter.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter.lean,Mathlib/Tactic/Linter/GenericSyntaxLinter.lean,test/GenericSyntaxLinter.lean |
7 |
19 |
['adomani', 'github-actions', 'grunweg', 'leanprover-bot'] |
nobody |
4-79521 4 days ago |
396-67656 1 year ago |
41-49960 41 days |
26908 |
robin-carlier author:robin-carlier |
feat(CategoryTheory/Monoidal/DayConvolution): alternative ext principle for unitors |
Currently, our infrastructure for left/right unitors for Day convolution of functors `C ⥤ V` do not have satisfactory extensionality principle: the current way to characterize morphisms out of `U ⊛ F` is the default extensionality principle for Day convolution, which characterizes first such functors via functors out of `U ⊠ F`. Left unitors are then obtained using the fact `U ⊠ F` is a left Kan extension of a functor from `PUnit × C` (which is equivalent to `C`) but we did not record on its own this principle.
Using the transitivity of left Kan extensions proved in #26899, we directly exhibit `U ⊛ F` as a left Kan extension of `F ⋙ tensorLeft (𝟙_ V)` along `tensorLeft (𝟙_ C)`. The unit of this Kan extension is composed exactly of the morphisms that appear in the [characterization of left unitors](https://leanprover-community.github.io/mathlib4_docs/Mathlib/CategoryTheory/Monoidal/DayConvolution.html#CategoryTheory.MonoidalCategory.DayConvolutionUnit.leftUnitor_hom_unit_app).
We also slightly generalize the instances that express that external products with unitors are left Kan extensions, so that they can be used when taking external products with more complicated functors than currently. This is again useful when chaining extensionality lemmas for morphisms out of terms of the form `(F ⊛ U) ⊛ G`.
We prove a similar thing for right unitors
With this, it should be possible to have a much more satisfactory way of working with Day convolutions: this allows to "elimiinate" units without ending up with terms in an external product.
---
- [ ] depends on: #26899
- [ ] depends on: #26906
[](https://gitpod.io/from-referrer/)
|
t-category-theory
merge-conflict
|
307/18 |
Mathlib/CategoryTheory/Functor/KanExtension/Basic.lean,Mathlib/CategoryTheory/Monoidal/DayConvolution.lean |
2 |
4 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
4-71214 4 days ago |
4-71215 4 days ago |
0-1812 30 minutes |
27150 |
robin-carlier author:robin-carlier |
feat(CategoryTheory/Monoidal/DayConvolution): constructors for braided and symmetric structure on day convolutions monoidal categories |
Following the pattern in #27119, we give API to construct `BraidedCategory` and `SymmetricCategory` structures on a monoidal
category equipped with a `LawfulDayConvolutionMonoidalCategoryStruct`. To achieve this, we introduce an other type class
`LawfulDayConvolutionBraidedCategoryStruct` that bundles an associator isomorphism that behaves like the one constructed for functors in #27067.
We provide a noncomputable constructor for this typeclass that takes as input fullness of the "realization" functor to a category of functors, and we show that the typeclasses are sufficient to define the desired structures.
---
- [x] depends on: #27067
- [x] depends on: #26820
[](https://gitpod.io/from-referrer/)
|
t-category-theory
merge-conflict
|
826/9 |
Mathlib/CategoryTheory/Monoidal/DayConvolution.lean,Mathlib/CategoryTheory/Monoidal/DayConvolution/Braided.lean |
2 |
5 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
4-66253 4 days ago |
4-67041 4 days ago |
0-1002 16 minutes |
26660 |
strihanje01 author:strihanje01 |
feat(Combinatorics/Additive/VerySmallDoubling): weak non-commutative Kneser's theorem |
add theorem about the structure of a doubling smaller than the golden ratio
---
- [ ] depends on: #28653
[](https://gitpod.io/from-referrer/)
|
large-import
new-contributor
t-combinatorics
merge-conflict
|
372/41 |
Mathlib.lean,Mathlib/Algebra/Group/Action/Pointwise/Finset.lean,Mathlib/Combinatorics/Additive/Convolution.lean,Mathlib/Combinatorics/Additive/VerySmallDoubling.lean |
4 |
75 |
['YaelDillies', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'strihanje01'] |
YaelDillies assignee:YaelDillies |
4-49541 4 days ago |
4-49541 4 days ago |
37-51670 37 days |
29390 |
harahu author:harahu |
doc(Computability): documentation improvement suggestions from Junie Pro (LLM) |
I'm still in the process of self-reviewing the details here, but please shout out if there are any changes you don't like.
---
[](https://gitpod.io/from-referrer/)
|
t-computability
merge-conflict
|
245/242 |
Mathlib/Computability/Ackermann.lean,Mathlib/Computability/AkraBazzi/AkraBazzi.lean,Mathlib/Computability/AkraBazzi/GrowsPolynomially.lean,Mathlib/Computability/AkraBazzi/SumTransform.lean,Mathlib/Computability/ContextFreeGrammar.lean,Mathlib/Computability/DFA.lean,Mathlib/Computability/Encoding.lean,Mathlib/Computability/EpsilonNFA.lean,Mathlib/Computability/Halting.lean,Mathlib/Computability/Language.lean,Mathlib/Computability/MyhillNerode.lean,Mathlib/Computability/NFA.lean,Mathlib/Computability/PartrecCode.lean,Mathlib/Computability/PostTuringMachine.lean,Mathlib/Computability/RegularExpressions.lean,Mathlib/Computability/TMComputable.lean,Mathlib/Computability/TMConfig.lean,Mathlib/Computability/TMToPartrec.lean,Mathlib/Computability/Tape.lean,Mathlib/Computability/TuringDegree.lean,Mathlib/Computability/TuringMachine.lean |
21 |
8 |
['github-actions', 'harahu'] |
nobody |
4-11333 4 days ago |
4-52025 4 days ago |
0-0 0 seconds |
27119 |
robin-carlier author:robin-carlier |
feat(CategoryTheory/Monoidal/DayConvolution): constructors for closed monoidal day convolution monoidal structures |
Following the pattern introduced in #26798 and #26820 and using results of #26879, we introduce a typeclass
`LawfulDayConvolutionClosedMonoidalCategoryStruct` that encodes the data needed on a `LawfulDayConvolutionMonoidalCategoryStruct` to define well-behaved internal homs. We give a constructor assuming existence of relevant ends, and prove that this data defines a `MonoidalClosed` instance on the monoidal category structures one can deduce from `LawfulDayConvolutionMonoidalCategoryStruct`.
---
- [x] depends on: #27079
- [x] depends on: #27091
- [x] depends on: #26879
- [x] depends on: #26820
[](https://gitpod.io/from-referrer/)
|
t-category-theory
merge-conflict
|
900/9 |
Mathlib/CategoryTheory/Monoidal/DayConvolution.lean,Mathlib/CategoryTheory/Monoidal/DayConvolution/Closed.lean |
2 |
6 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
3-80104 3 days ago |
4-67038 4 days ago |
0-1 1 second |
28411 |
zcyemi author:zcyemi |
feat(LinearAlgebra/AffineSpace/Simplex/Centroid): define centroid and medians |
---
This file proves several lemmas involving the centroids and medians of a simplex in affine space.
definitions:
- `centroid` is the centroid of a simplex, defined as abbreviation of the `Finset.univ.centroid`.
- `faceOppositeCentroid` is the centroid of the facet obtained as `(Simplex.faceOpposite i).centroid`
- `median` is the line connecting a vertex to the faceOppositeCentroid.
Main Results:
- Commandino's theorem
- The medians of a simplex are concurrent at the centroid
- [ ] depends on #29128 |
large-import
t-algebra
merge-conflict
label:t-algebra$ |
463/5 |
Mathlib/Geometry/Euclidean/MongePoint.lean,Mathlib/Geometry/Euclidean/Simplex.lean,Mathlib/LinearAlgebra/AffineSpace/Independent.lean,Mathlib/LinearAlgebra/AffineSpace/Simplex/Centroid.lean,docs/1000.yaml |
5 |
9 |
['github-actions', 'jsm28', 'mathlib4-merge-conflict-bot', 'zcyemi'] |
nobody |
3-74089 3 days ago |
3-74090 3 days ago |
25-79919 25 days |
28623 |
gilesgshaw author:gilesgshaw |
feat(Logic/Basic): minor additions and simplification of proofs |
Add new theorems and simplify proofs.
Specifically, we add the family of related theorems `apply_dite_iff_exists`, `apply_dite_iff_forall`, `apply_ite_iff_and` and `apply_ite_iff_or`.
For each other 'family' of theorems in the file that is analogous to the above, we do the following
- Simplify proofs where possible, e.g. by appealing to the new theorems
- Complete the family, if any of the corresponding four are missing
- Rename to ensure consistency with the above pattern
---
|
new-contributor
t-logic
merge-conflict
|
83/55 |
Archive/Examples/IfNormalization/Result.lean,Archive/Examples/IfNormalization/WithoutAesop.lean,Mathlib/Algebra/ContinuedFractions/Computation/Translations.lean,Mathlib/Algebra/MvPolynomial/Variables.lean,Mathlib/Algebra/Notation/Indicator.lean,Mathlib/LinearAlgebra/Matrix/Rank.lean,Mathlib/Logic/Basic.lean,Mathlib/MeasureTheory/Measure/WithDensity.lean,Mathlib/SetTheory/Ordinal/Notation.lean |
9 |
12 |
['eric-wieser', 'gilesgshaw', 'github-actions', 'mathlib4-merge-conflict-bot', 'plp127'] |
awainverse assignee:awainverse |
3-73965 3 days ago |
3-73966 3 days ago |
21-3001 21 days |
24692 |
ScottCarnahan author:ScottCarnahan |
feat (RingTheory/HahnSeries/Basic): isomorphism of Hahn series induced by order isomorphism |
This PR introduces an isomorphism of Hahn series induced by an order isomorphism on the exponent posets.
---
[](https://gitpod.io/from-referrer/)
|
t-order
merge-conflict
WIP
|
35/0 |
Mathlib/RingTheory/HahnSeries/Basic.lean |
1 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
3-50345 3 days ago |
3-50346 3 days ago |
31-47622 31 days |
25822 |
ScottCarnahan author:ScottCarnahan |
WIP: experiments with vertex algebras |
This is a testbed for various attempts at things. Please don't bother reviewing.
---
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #25821.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/25821* |
large-import
merge-conflict
WIP
|
7726/332 |
Mathlib.lean,Mathlib/Algebra/Group/Action/Basic.lean,Mathlib/Algebra/Lie/ChevalleyEilenberg.lean,Mathlib/Algebra/Lie/Cocycle.lean,Mathlib/Algebra/Lie/Extension.lean,Mathlib/Algebra/Lie/Extension/Basic.lean,Mathlib/Algebra/Lie/Extension/CentralExtension.lean,Mathlib/Algebra/Lie/Loop.lean,Mathlib/Algebra/Module/Equiv/Basic.lean,Mathlib/Algebra/Module/Equiv/Defs.lean,Mathlib/Algebra/Order/AddTorsor.lean,Mathlib/Algebra/Order/Monoid/Prod.lean,Mathlib/Algebra/Polynomial/Laurent.lean,Mathlib/Algebra/Polynomial/Nusmeval.lean,Mathlib/Algebra/Polynomial/Smeval.lean,Mathlib/Algebra/Vertex/Affine.lean,Mathlib/Algebra/Vertex/Basic.lean,Mathlib/Algebra/Vertex/Defs.lean,Mathlib/Algebra/Vertex/HVertexOperator.lean,Mathlib/Algebra/Vertex/VertexOperator.lean,Mathlib/Data/Finset/SMulAntidiagonal.lean,Mathlib/Data/Finsupp/PointwiseSMul.lean,Mathlib/Data/FunLike/Equiv.lean,Mathlib/Data/Prod/RevLex.lean,Mathlib/Data/Set/SMulAntidiagonal.lean,Mathlib/GroupTheory/GroupAction/Equiv.lean,Mathlib/GroupTheory/GroupAction/Hom.lean,Mathlib/RingTheory/Binomial.lean,Mathlib/RingTheory/DividedPowers/Cauchy.lean,Mathlib/RingTheory/FormalSeries.lean,Mathlib/RingTheory/HahnSeries/Addition.lean,Mathlib/RingTheory/HahnSeries/Basic.lean,Mathlib/RingTheory/HahnSeries/Binomial.lean,Mathlib/RingTheory/HahnSeries/HEval.lean,Mathlib/RingTheory/HahnSeries/Multiplication.lean,Mathlib/RingTheory/HahnSeries/PowerSeries.lean,Mathlib/RingTheory/HahnSeries/Summable.lean,Mathlib/RingTheory/LaurentSeries.lean,Mathlib/RingTheory/PowerSeries/Binomial.lean,Mathlib/RingTheory/PowerSeries/Eval.lean |
40 |
n/a |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-merge-conflict-bot'] |
nobody |
3-50040 3 days ago |
unknown |
unknown |
29061 |
chrisflav author:chrisflav |
refactor(AlgebraicGeometry): replace `Scheme.Cover` by an `abbrev` for `ZeroHypercover` |
We replace `Scheme.Cover` by an `abbrev` for `Coverage.ZeroHypercover`. The main motivation is to allow for a generalization of `IsLocalAtTarget`, `IsLocalAtSource` etc. to arbitrary coverages. The second motivation is to reduce duplication in the upcoming introduction of categories of analytic spaces (e.g. adic spaces), by generalizing notions of `Cover` to suitable general categories.
The main (breaking) API change is that the fields of `Cover` are now called differently:
- `obj → X`
- `map → f`
- `J → I₀`.
For reducing the diff in this refactor, we keep `abbrev`s for the old names. These shall be deprecated in a follow-up PR.
Future work: Besides the generalisation of `IsLocalAtTarget`, the content of `AlgebraicGeometry.Cover.Over` and `AlgebraicGeometry.Sites.Small` shall be generalized to general coverages instead of the coverage induced by a morphism property.
---
- [x] depends on: #28778
- [x] depends on: #29065
- [ ] depends on: #29467
This PR will be split in more reviewable pieces when agreement is reached on the general direction this PR is taking.
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebraic-geometry
merge-conflict
|
1120/969 |
Mathlib.lean,Mathlib/AlgebraicGeometry/AffineScheme.lean,Mathlib/AlgebraicGeometry/AffineSpace.lean,Mathlib/AlgebraicGeometry/Cover/Directed.lean,Mathlib/AlgebraicGeometry/Cover/MorphismProperty.lean,Mathlib/AlgebraicGeometry/Cover/Open.lean,Mathlib/AlgebraicGeometry/Cover/Over.lean,Mathlib/AlgebraicGeometry/Cover/Sigma.lean,Mathlib/AlgebraicGeometry/FunctionField.lean,Mathlib/AlgebraicGeometry/Gluing.lean,Mathlib/AlgebraicGeometry/GluingOneHypercover.lean,Mathlib/AlgebraicGeometry/IdealSheaf/Basic.lean,Mathlib/AlgebraicGeometry/IdealSheaf/Subscheme.lean,Mathlib/AlgebraicGeometry/Limits.lean,Mathlib/AlgebraicGeometry/Morphisms/Basic.lean,Mathlib/AlgebraicGeometry/Morphisms/Constructors.lean,Mathlib/AlgebraicGeometry/Morphisms/FinitePresentation.lean,Mathlib/AlgebraicGeometry/Morphisms/FiniteType.lean,Mathlib/AlgebraicGeometry/Morphisms/LocalClosure.lean,Mathlib/AlgebraicGeometry/Morphisms/QuasiCompact.lean,Mathlib/AlgebraicGeometry/Morphisms/QuasiSeparated.lean,Mathlib/AlgebraicGeometry/Morphisms/RingHomProperties.lean,Mathlib/AlgebraicGeometry/Morphisms/Separated.lean,Mathlib/AlgebraicGeometry/Morphisms/SurjectiveOnStalks.lean,Mathlib/AlgebraicGeometry/Morphisms/UnderlyingMap.lean,Mathlib/AlgebraicGeometry/Morphisms/UniversallyClosed.lean,Mathlib/AlgebraicGeometry/Noetherian.lean,Mathlib/AlgebraicGeometry/PointsPi.lean,Mathlib/AlgebraicGeometry/ProjectiveSpectrum/Basic.lean,Mathlib/AlgebraicGeometry/Properties.lean,Mathlib/AlgebraicGeometry/Pullbacks.lean,Mathlib/AlgebraicGeometry/RationalMap.lean,Mathlib/AlgebraicGeometry/Restrict.lean,Mathlib/AlgebraicGeometry/Sites/BigZariski.lean,Mathlib/AlgebraicGeometry/Sites/MorphismProperty.lean,Mathlib/AlgebraicGeometry/Sites/Pretopology.lean,Mathlib/AlgebraicGeometry/Sites/Representability.lean,Mathlib/AlgebraicGeometry/Sites/Small.lean,Mathlib/AlgebraicGeometry/SpreadingOut.lean,Mathlib/AlgebraicGeometry/Stalk.lean,Mathlib/CategoryTheory/Sites/Sieves.lean,Mathlib/CategoryTheory/Sites/ZeroHypercover.lean |
42 |
4 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
3-37883 3 days ago |
3-37884 3 days ago |
0-11046 3 hours |
29461 |
kim-em author:kim-em |
wip: grind/omega |
Context: `omega` is poorly implemented, and we'd eventually like to deprecate it outside of bootstrapping Lean itself. Currently `grind` is only a partial replacement, but we're working on getting it to parity.
This PR replaces all the occurrences of `omega` which can be replaced by `grind` today. Note that overall there is a slight reduction in the total instruction count for building Mathlib (despite increases in certain files). So my preference is to not worry about the performance side of things here. (I've split the PR into two commits: the first commit contains only changes which do not introduce even a local slow-down. The second commit contains the ~25 files which have a local performance penalty.) Even the file with the most significant slowdown, Mathlib.RingTheory.AdicCompletion.Exactness, seems perfectly fine in VSCode to me.
There is separately the valid question about the readability of proofs: is it sometimes helpful to know that the problem can be solved by the omega algorithm? (Note that `grind` uses a completely different algorithm for this class of problems.) We could provide a `cutsat` frontend for `grind`, which disables nearly everything except the cutsat solver. This would then preserve the information in the proof script that "it's only a linear integer arithmetic (+ lots of fancy preprocessing) problem". |
merge-conflict |
1960/1958 |
Archive/Imo/Imo1960Q1.lean,Archive/Imo/Imo1962Q1.lean,Archive/Imo/Imo1985Q2.lean,Archive/Imo/Imo1988Q6.lean,Archive/Imo/Imo1994Q1.lean,Archive/Imo/Imo1997Q3.lean,Archive/Imo/Imo2001Q3.lean,Archive/Imo/Imo2001Q6.lean,Archive/Imo/Imo2008Q3.lean,Archive/Imo/Imo2015Q6.lean,Archive/Imo/Imo2021Q1.lean,Archive/Imo/Imo2024Q1.lean,Archive/Imo/Imo2024Q2.lean,Archive/Imo/Imo2024Q3.lean,Archive/Imo/Imo2024Q5.lean,Archive/Wiedijk100Theorems/AscendingDescendingSequences.lean,Archive/Wiedijk100Theorems/FriendshipGraphs.lean,Counterexamples/AharoniKorman.lean,Counterexamples/DiscreteTopologyNonDiscreteUniformity.lean,Mathlib/Algebra/AddConstMap/Basic.lean,Mathlib/Algebra/BigOperators/Fin.lean,Mathlib/Algebra/BigOperators/Intervals.lean,Mathlib/Algebra/ContinuedFractions/Computation/Approximations.lean,Mathlib/Algebra/ContinuedFractions/Computation/TerminatesIffRat.lean,Mathlib/Algebra/CubicDiscriminant.lean,Mathlib/Algebra/GCDMonoid/Nat.lean,Mathlib/Algebra/Group/Defs.lean,Mathlib/Algebra/Group/Fin/Basic.lean,Mathlib/Algebra/Group/Int/Even.lean,Mathlib/Algebra/Group/Int/Units.lean,Mathlib/Algebra/Group/Nat/Even.lean,Mathlib/Algebra/Group/Nat/Range.lean,Mathlib/Algebra/GroupWithZero/Basic.lean,Mathlib/Algebra/GroupWithZero/Units/Basic.lean,Mathlib/Algebra/Homology/ComplexShapeSigns.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/Basic.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/EnoughInjectives.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/EnoughProjectives.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/ExactSequences.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/ExtClass.lean,Mathlib/Algebra/Homology/DerivedCategory/Fractions.lean,Mathlib/Algebra/Homology/DerivedCategory/TStructure.lean,Mathlib/Algebra/Homology/Embedding/AreComplementary.lean,Mathlib/Algebra/Homology/Embedding/Basic.lean,Mathlib/Algebra/Homology/Embedding/Boundary.lean,Mathlib/Algebra/Homology/Embedding/CochainComplex.lean,Mathlib/Algebra/Homology/Embedding/Connect.lean,Mathlib/Algebra/Homology/ExactSequence.lean,Mathlib/Algebra/Homology/HomotopyCategory/DegreewiseSplit.lean,Mathlib/Algebra/Homology/HomotopyCategory/HomComplex.lean,Mathlib/Algebra/Homology/HomotopyCategory/HomComplexShift.lean,Mathlib/Algebra/Homology/HomotopyCategory/MappingCone.lean,Mathlib/Algebra/Homology/HomotopyCategory/Pretriangulated.lean,Mathlib/Algebra/Homology/HomotopyCategory/Shift.lean,Mathlib/Algebra/Homology/HomotopyCategory/ShiftSequence.lean,Mathlib/Algebra/Homology/HomotopyCategory/ShortExact.lean,Mathlib/Algebra/Homology/HomotopyCategory/SingleFunctors.lean,Mathlib/Algebra/Homology/HomotopyCategory/Triangulated.lean,Mathlib/Algebra/Homology/TotalComplexShift.lean,Mathlib/Algebra/Lie/CartanExists.lean,Mathlib/Algebra/Lie/EngelSubalgebra.lean,Mathlib/Algebra/Lie/LieTheorem.lean,Mathlib/Algebra/Lie/Nilpotent.lean,Mathlib/Algebra/Lie/Sl2.lean,Mathlib/Algebra/Lie/Weights/Chain.lean,Mathlib/Algebra/Lie/Weights/Killing.lean,Mathlib/Algebra/Lie/Weights/RootSystem.lean,Mathlib/Algebra/LinearRecurrence.lean,Mathlib/Algebra/ModEq.lean,Mathlib/Algebra/Module/LinearMap/End.lean,Mathlib/Algebra/MvPolynomial/Degrees.lean,Mathlib/Algebra/Order/Antidiag/Nat.lean,Mathlib/Algebra/Order/CauSeq/BigOperators.lean,Mathlib/Algebra/Order/Floor/Ring.lean,Mathlib/Algebra/Order/Group/Basic.lean,Mathlib/Algebra/Order/Group/DenselyOrdered.lean,Mathlib/Algebra/Order/Group/Int/Sum.lean,Mathlib/Algebra/Order/Group/Unbundled/Int.lean,Mathlib/Algebra/Order/GroupWithZero/Unbundled/Basic.lean,Mathlib/Algebra/Order/Monoid/Unbundled/Pow.lean,Mathlib/Algebra/Order/Ring/GeomSum.lean,Mathlib/Algebra/Order/Ring/Int.lean,Mathlib/Algebra/Order/Ring/Unbundled/Rat.lean,Mathlib/Algebra/Polynomial/AlgebraMap.lean,Mathlib/Algebra/Polynomial/CoeffList.lean,Mathlib/Algebra/Polynomial/Degree/CardPowDegree.lean,Mathlib/Algebra/Polynomial/Degree/IsMonicOfDegree.lean,Mathlib/Algebra/Polynomial/Derivative.lean,Mathlib/Algebra/Polynomial/FieldDivision.lean,Mathlib/Algebra/Polynomial/Laurent.lean,Mathlib/Algebra/Polynomial/OfFn.lean,Mathlib/Algebra/Polynomial/Sequence.lean,Mathlib/Algebra/Ring/Divisibility/Lemmas.lean,Mathlib/Algebra/Ring/GeomSum.lean,Mathlib/Algebra/Ring/Parity.lean,Mathlib/Algebra/Squarefree/Basic.lean,Mathlib/Algebra/Vertex/VertexOperator.lean,Mathlib/AlgebraicGeometry/EllipticCurve/DivisionPolynomial/Degree.lean,Mathlib/AlgebraicGeometry/ProjectiveSpectrum/Scheme.lean,Mathlib/AlgebraicGeometry/StructureSheaf.lean |
470 |
6 |
['github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
3-15861 3 days ago |
3-15862 3 days ago |
0-0 0 seconds |
28737 |
astrainfinita author:astrainfinita |
refactor: deprecate `MulEquivClass` |
This PR continues the work from #18806.
Original PR: https://github.com/leanprover-community/mathlib4/pull/18806 |
maintainer-merge
t-algebra
merge-conflict
awaiting-author
label:t-algebra$ |
67/77 |
Mathlib/Algebra/BigOperators/Finprod.lean,Mathlib/Algebra/Group/Equiv/Basic.lean,Mathlib/Algebra/Group/Equiv/Defs.lean,Mathlib/Algebra/Group/Irreducible/Lemmas.lean,Mathlib/Algebra/Group/Subgroup/Map.lean,Mathlib/Algebra/Group/Submonoid/Operations.lean,Mathlib/Algebra/Group/Units/Equiv.lean,Mathlib/Algebra/GroupWithZero/Equiv.lean,Mathlib/Algebra/GroupWithZero/NonZeroDivisors.lean,Mathlib/Algebra/Module/Equiv/Defs.lean,Mathlib/Algebra/Order/CauSeq/Basic.lean,Mathlib/Algebra/Order/Hom/Monoid.lean,Mathlib/Algebra/Prime/Lemmas.lean,Mathlib/Algebra/Ring/Divisibility/Basic.lean,Mathlib/Algebra/Ring/Equiv.lean,Mathlib/Algebra/Star/MonoidHom.lean,Mathlib/Combinatorics/Additive/FreimanHom.lean,Mathlib/GroupTheory/GroupExtension/Defs.lean,Mathlib/GroupTheory/Submonoid/Center.lean,Mathlib/LinearAlgebra/FreeModule/Finite/CardQuotient.lean,Mathlib/RingTheory/Bialgebra/Equiv.lean,Mathlib/RingTheory/Ideal/Norm/AbsNorm.lean,Mathlib/RingTheory/Multiplicity.lean,Mathlib/RingTheory/UniqueFactorizationDomain/NormalizedFactors.lean,Mathlib/Topology/Algebra/ContinuousMonoidHom.lean,Mathlib/Topology/Algebra/InfiniteSum/Basic.lean |
26 |
20 |
['Vierkantor', 'alreadydone', 'astrainfinita', 'github-actions', 'grunweg', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'mathlib4-merge-conflict-bot'] |
Vierkantor assignee:Vierkantor |
2-80689 2 days ago |
2-80690 2 days ago |
4-17723 4 days |
28944 |
linesthatinterlace author:linesthatinterlace |
refactor(Order/Hom/Basic): reorder definitions |
Reorder and disentangle definitions for OrderHom, OrderEmbedding and OrderIso.
---
This is a preamble to making all of these `def` and consistently defined - the aim is to first disentangle the definitions as it will make it more straightforward to perform these later PRs.
[](https://gitpod.io/from-referrer/)
|
t-order
merge-conflict
|
217/188 |
Mathlib/Order/FixedPoints.lean,Mathlib/Order/Hom/Basic.lean,Mathlib/Order/Hom/Order.lean |
3 |
6 |
['YaelDillies', 'github-actions', 'linesthatinterlace', 'mathlib4-merge-conflict-bot'] |
YaelDillies, b-mehta, linesthatinterlace assignee:YaelDillies assignee:b-mehta assignee:linesthatinterlace |
2-64503 2 days ago |
2-64504 2 days ago |
15-28022 15 days |
27284 |
FernandoChu author:FernandoChu |
Chore(CategoryTheory/MorphismProperty/MonoFactorization): Factor out mono factorizations |
Factored out `MonoFactorisations` from the `Images` file; also rename it to `MonoFactori*z*ations` so it's inline with the rest of Mathlib. I'm also sneaking in some very basic extremal epis results if you don't mind, these were meant to be used to prove
```lean
instance (priority := 100) hasStrongEpiImages_of_hasPullbacks_of_hasEqualizers [HasPullbacks C]
[HasEqualizers C] : HasStrongEpiImages C
```
Which I noticed too late already had a proof; I think the proof has been improved anyways, it's just `infer_instance` now. |
new-contributor
t-category-theory
merge-conflict
awaiting-author
|
489/311 |
Mathlib.lean,Mathlib/Algebra/Category/Grp/Images.lean,Mathlib/Algebra/Category/ModuleCat/Images.lean,Mathlib/AlgebraicTopology/SimplexCategory/Basic.lean,Mathlib/CategoryTheory/Abelian/Basic.lean,Mathlib/CategoryTheory/Category/Factorisation.lean,Mathlib/CategoryTheory/ConcreteCategory/EpiMono.lean,Mathlib/CategoryTheory/Limits/Preserves/Shapes/Images.lean,Mathlib/CategoryTheory/Limits/Shapes/ExtremalEpi.lean,Mathlib/CategoryTheory/Limits/Shapes/Images.lean,Mathlib/CategoryTheory/Limits/Shapes/Kernels.lean,Mathlib/CategoryTheory/Limits/Shapes/StrongEpi.lean,Mathlib/CategoryTheory/Limits/Shapes/ZeroMorphisms.lean,Mathlib/CategoryTheory/Limits/Types/Images.lean,Mathlib/CategoryTheory/MorphismProperty/MonoFactorization.lean,Mathlib/CategoryTheory/Sites/Subsheaf.lean,Mathlib/Order/Category/NonemptyFinLinOrd.lean,scripts/nolints_prime_decls.txt |
18 |
46 |
['FernandoChu', 'Ruben-VandeVelde', 'bryangingechen', 'github-actions', 'joelriou', 'mathlib4-merge-conflict-bot', 'robin-carlier'] |
nobody |
2-61903 2 days ago |
2-61904 2 days ago |
16-75072 16 days |
29364 |
hrmacbeth author:hrmacbeth |
feat(Tactic/FieldSimp): handle inequalities |
---
[](https://gitpod.io/from-referrer/)
|
large-import
merge-conflict
|
214/78 |
Mathlib/Analysis/Calculus/BumpFunction/FiniteDimension.lean,Mathlib/Analysis/Convex/Continuous.lean,Mathlib/Analysis/Convex/Mul.lean,Mathlib/Analysis/Convex/Slope.lean,Mathlib/Analysis/PSeries.lean,Mathlib/Analysis/SpecialFunctions/Stirling.lean,Mathlib/RingTheory/RootsOfUnity/Complex.lean,Mathlib/Tactic/FieldSimp.lean,Mathlib/Tactic/FieldSimp/Lemmas.lean |
9 |
3 |
['github-actions', 'grunweg', 'mathlib4-merge-conflict-bot'] |
nobody |
2-53157 2 days ago |
2-57214 2 days ago |
0-0 0 seconds |
13036 |
joelriou author:joelriou |
feat(CategoryTheory/Sites): under certain conditions, cover preserving functors preserve 1-hypercovers |
Previously, in order to show that a functor between Grothendieck sites was continuous, it was necessary to show that it was "cover preserving" and "compatible preserving". There were two lemmas which could be used in order to show that a functor was "compatible preserving".
Since #13012, the better condition of "1-hypercover preserving" functor was introduced and it implies that the functor is continuous. In this PR, under the same assumptions as in the two lemmas mentionned above, we show that cover preserving functors are 1-hypercover preserving functors. This gives slightly better criteria in order to show that a functor is continuous.
---
- [x] depends on: #13004
- [x] depends on: #13011
- [x] depends on: #13012
[](https://gitpod.io/from-referrer/)
|
t-category-theory
merge-conflict
WIP
|
94/7 |
Mathlib/CategoryTheory/Sites/Continuous.lean,Mathlib/CategoryTheory/Sites/CoverPreserving.lean,Mathlib/CategoryTheory/Sites/Over.lean,Mathlib/CategoryTheory/Sites/Sieves.lean |
4 |
3 |
['github-actions', 'leanprover-community-mathlib4-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
2-43289 2 days ago |
2-43290 2 days ago |
0-0 0 seconds |
27335 |
eric-wieser author:eric-wieser |
chore(Data/List): use simp-normal-form for boolean equalities |
This replaces `¬(p x = true)` with `p x = false`. It also makes explicit some adjacent `h : p x` spellings for symmetry, but the `= true`s were already implied by the coercion.
Zulip: [#lean4 > `h : ¬(b = true)` vs `h : b = false` @ 💬](https://leanprover.zulipchat.com/#narrow/channel/270676-lean4/topic/.60h.20.3A.20.C2.AC.28b.20.3D.20true.29.60.20vs.20.60h.20.3A.20b.20.3D.20false.60/near/529976237)
---
[](https://gitpod.io/from-referrer/)
|
t-data
merge-conflict
|
38/32 |
Mathlib/Data/List/DropRight.lean,Mathlib/Data/List/SplitOn.lean,Mathlib/Data/List/TakeWhile.lean |
3 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-merge-conflict-bot'] |
nobody |
2-26931 2 days ago |
2-26932 2 days ago |
4-31215 4 days |
21965 |
JovanGerb author:JovanGerb |
feat: extensible `push` and `pull` tactics |
This PR defines the `push` and `pull` tactics, and makes `push_neg` a macro for `push Not`. The tactics are also available in `conv` mode.
For tagging, there is only the `@[push]` attribute, which adds the reverse rewrite for the `pull` tactic when relevant. In the future, we may also need a separate `@[pull X]` attribute for pulling `X`.
Thanks to this change, we will be able to make `push_neg` into a more powerful tactic by tagging more lemmas. It also means that about 60 files now don't need to import `LinearOrder`/`PartialOrder`. This will be especially useful when we get the `@[to_dual]` attribute.
This work originally started in #21769. There is now the follow up PR #29000 which adds `push` tags and tests for them.
The `@[push]` attribute is defined in `Mathlib.Tactic.Push.Attr` and the main implementation of `push` and `pull` is in `Mathlib.Tactic.Push`.
Some proofs need to be fixed because the new simp-based `push_neg` can see through more reducible definitions.
Zulip conversation: [#mathlib4 > I made an extensible `push` tactic generalizing `push_neg`](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/I.20made.20an.20extensible.20.60push.60.20tactic.20generalizing.20.60push_neg.60)
closes #21841
---
[](https://gitpod.io/from-referrer/)
|
maintainer-merge
t-meta
merge-conflict
|
505/178 |
Mathlib.lean,Mathlib/Algebra/Lie/Weights/Killing.lean,Mathlib/Combinatorics/SimpleGraph/Coloring.lean,Mathlib/Combinatorics/SimpleGraph/Extremal/Basic.lean,Mathlib/Data/Nat/Basic.lean,Mathlib/Data/Set/Basic.lean,Mathlib/Order/Defs/LinearOrder.lean,Mathlib/RingTheory/AlgebraicIndependent/TranscendenceBasis.lean,Mathlib/RingTheory/HahnSeries/Lex.lean,Mathlib/RingTheory/Multiplicity.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Push.lean,Mathlib/Tactic/Push/Attr.lean,Mathlib/Topology/Algebra/IsUniformGroup/Basic.lean,MathlibTest/push.lean,MathlibTest/push_neg.lean,scripts/noshake.json |
17 |
62 |
['JovanGerb', 'adomani', 'github-actions', 'grunweg', 'j-loreaux', 'leanprover-bot', 'leanprover-community-bot-assistant', 'mathlib4-merge-conflict-bot', 'plp127'] |
robertylewis assignee:robertylewis |
2-21687 2 days ago |
2-21688 2 days ago |
138-79638 138 days |
28241 |
alreadydone author:alreadydone |
chore(Data): `SetLike Finset` |
---
[](https://gitpod.io/from-referrer/)
|
t-data
merge-conflict
|
54/62 |
Counterexamples/AharoniKorman.lean,Mathlib/Algebra/BigOperators/Finprod.lean,Mathlib/Algebra/Group/Pointwise/Finset/Basic.lean,Mathlib/Algebra/Module/FinitePresentation.lean,Mathlib/Combinatorics/Additive/RuzsaCovering.lean,Mathlib/Combinatorics/SimpleGraph/Connectivity/WalkCounting.lean,Mathlib/Data/DFinsupp/Defs.lean,Mathlib/Data/Finset/Defs.lean,Mathlib/Data/Finset/Insert.lean,Mathlib/Data/Finset/Union.lean,Mathlib/FieldTheory/Perfect.lean,Mathlib/GroupTheory/Perm/Centralizer.lean,Mathlib/GroupTheory/Perm/Cycle/Basic.lean,Mathlib/LinearAlgebra/Finsupp/LinearCombination.lean,Mathlib/LinearAlgebra/Finsupp/Supported.lean,Mathlib/LinearAlgebra/LinearIndependent/Basic.lean,Mathlib/LinearAlgebra/LinearIndependent/Defs.lean,Mathlib/MeasureTheory/Integral/IntegrableOn.lean,Mathlib/ModelTheory/Semantics.lean,Mathlib/Order/CountableDenseLinearOrder.lean,Mathlib/Probability/Independence/Kernel.lean,Mathlib/RingTheory/Ideal/Quotient/Index.lean,Mathlib/RingTheory/IntegralClosure/IsIntegral/Basic.lean,Mathlib/RingTheory/Spectrum/Prime/Polynomial.lean,Mathlib/Topology/Separation/Basic.lean |
25 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
2-20008 2 days ago |
2-20009 2 days ago |
29-66463 29 days |
29442 |
Vierkantor author:Vierkantor |
chore(*): replace remaining `simp? says` with `simp only` |
For the cases where the previous PRs (#29440, #29441) would not result in a nice to read proof, replace the output of `simp? says` with a `simp only`, and then golf the result by trying to drop lemmas from the simp set, or even replace it outright with (`simp_`)`rw`.
If we go from `simp? [foo] says simp only [foo]` to `simp only [foo]` this seems like an improvement, or if we end up with a small set of `simp only` arguments, I think this is a clear win. And for the other cases, removing a relatively fragile mechanism of `simp? says` seems to be enough of a win to offset the large block of `simp only` arguments.
Zulip thread: https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/noisy.20simp.20says.20in.20CI
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict |
75/101 |
Archive/Examples/IfNormalization/Result.lean,Archive/Examples/IfNormalization/WithoutAesop.lean,Mathlib/Algebra/Homology/Augment.lean,Mathlib/Algebra/Homology/BifunctorHomotopy.lean,Mathlib/Algebra/MvPolynomial/Rename.lean,Mathlib/Algebra/Polynomial/Coeff.lean,Mathlib/AlgebraicTopology/SimplexCategory/Basic.lean,Mathlib/Analysis/Calculus/ContDiff/FaaDiBruno.lean,Mathlib/Analysis/Calculus/IteratedDeriv/FaaDiBruno.lean,Mathlib/CategoryTheory/GuitartExact/VerticalComposition.lean,Mathlib/CategoryTheory/Limits/FilteredColimitCommutesFiniteLimit.lean,Mathlib/CategoryTheory/Limits/Shapes/NormalMono/Equalizers.lean,Mathlib/CategoryTheory/Monoidal/Braided/Transport.lean,Mathlib/CategoryTheory/Products/Basic.lean,Mathlib/Computability/PartrecCode.lean,Mathlib/Computability/TMToPartrec.lean,Mathlib/Data/Fin/SuccPred.lean,Mathlib/Data/Finset/NoncommProd.lean,Mathlib/Data/List/Sigma.lean,Mathlib/Data/Ordmap/Ordset.lean,Mathlib/Data/PFunctor/Multivariate/M.lean,Mathlib/Data/QPF/Multivariate/Constructions/Fix.lean,Mathlib/Data/Seq/Parallel.lean,Mathlib/Data/Set/Enumerate.lean,Mathlib/Data/WSeq/Basic.lean,Mathlib/Data/WSeq/Productive.lean,Mathlib/Data/WSeq/Relation.lean,Mathlib/Geometry/Manifold/Instances/Icc.lean,Mathlib/GroupTheory/CoprodI.lean,Mathlib/MeasureTheory/Integral/Lebesgue/Add.lean,Mathlib/NumberTheory/Zsqrtd/Basic.lean,Mathlib/Tactic/NormNum/Ineq.lean |
32 |
3 |
['github-actions', 'grunweg', 'mathlib4-merge-conflict-bot'] |
nobody |
1-83839 1 day ago |
1-83840 1 day ago |
2-67515 2 days |
29499 |
chrisflav author:chrisflav |
feat(CategoryTheory/Sites): sheafification via hypercovers |
This is very much WIP, but I need a fresh cache.
---
[](https://gitpod.io/from-referrer/)
|
t-category-theory
merge-conflict
WIP
|
2121/1 |
Mathlib.lean,Mathlib/CategoryTheory/Sites/HomotopyOneHypercover.lean,Mathlib/CategoryTheory/Sites/Hypercover/Refinement.lean,Mathlib/CategoryTheory/Sites/Hypercover/Sheafification.lean,Mathlib/CategoryTheory/Sites/OneHypercover.lean,Mathlib/CategoryTheory/Sites/ZeroHypercover.lean |
6 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
1-83837 1 day ago |
1-83838 1 day ago |
0-0 0 seconds |
29484 |
eric-wieser author:eric-wieser |
refactor: switch to [] notation for Stream' |
I'll continue fixing this only if people agree this is a good use of this notation.
[#mathlib4 > Changing `Stream.Seq` to use `GetElem` @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Changing.20.60Stream.2ESeq.60.20to.20use.20.60GetElem.60/near/538548680)
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-data
merge-conflict
|
195/173 |
Mathlib/Algebra/ContinuedFractions/Basic.lean,Mathlib/Algebra/ContinuedFractions/Computation/Basic.lean,Mathlib/Algebra/ContinuedFractions/Translations.lean,Mathlib/Combinatorics/Hindman.lean,Mathlib/Control/Fix.lean,Mathlib/Control/LawfulFix.lean,Mathlib/Data/Seq/Computation.lean,Mathlib/Data/Seq/Defs.lean,Mathlib/Data/Stream/Defs.lean,Mathlib/Data/Stream/Init.lean,Mathlib/Data/WSeq/Basic.lean,Mathlib/Data/WSeq/Productive.lean |
12 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
1-41950 1 day ago |
1-83839 1 day ago |
0-0 0 seconds |
29143 |
RemyDegenne author:RemyDegenne |
feat(Probability/Decision): basic properties of the Bayes risk |
- Comparison of the Bayes risk and the minimax risk
- Maximal value of the Bayes risk and particular cases where it equals that value
- Data-processing inequality
---
- [ ] depends on: #29137
[](https://gitpod.io/from-referrer/)
|
t-measure-probability
merge-conflict
|
276/17 |
Mathlib.lean,Mathlib/Probability/Decision/Risk/Basic.lean,Mathlib/Probability/Kernel/Composition/Comp.lean,Mathlib/Probability/Kernel/Composition/MapComap.lean,Mathlib/Probability/Kernel/Defs.lean,Mathlib/Probability/Kernel/RadonNikodym.lean |
6 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
0-63060 17 hours ago |
0-63061 17 hours ago |
0-5222 1 hour |
26138 |
xroblot author:xroblot |
Development branch (2) |
---
[](https://gitpod.io/from-referrer/)
|
large-import
merge-conflict
WIP
|
4643/179 |
Mathlib.lean,Mathlib/Algebra/Group/Opposite.lean,Mathlib/Algebra/Group/Torsion.lean,Mathlib/Algebra/Polynomial/Eval/Degree.lean,Mathlib/Algebra/Ring/NonZeroDivisors.lean,Mathlib/Basis.lean,Mathlib/Cyclotomic.lean,Mathlib/Discriminant.lean,Mathlib/FieldTheory/Galois/Basic.lean,Mathlib/FieldTheory/IntermediateField/Basic.lean,Mathlib/FieldTheory/LinearDisjoint.lean,Mathlib/Inertia.lean,Mathlib/LinearAlgebra/BilinearForm/Properties.lean,Mathlib/Misc.lean,Mathlib/NumberTheory/NumberField/Discriminant/Defs.lean,Mathlib/NumberTheory/NumberField/Discriminant/Different.lean,Mathlib/NumberTheory/RamificationInertia/Basic.lean,Mathlib/RingTheory/Binomial.lean,Mathlib/RingTheory/DedekindDomain/Different.lean,Mathlib/RingTheory/DedekindDomain/Factorization.lean,Mathlib/RingTheory/DedekindDomain/Ideal/Basic.lean,Mathlib/RingTheory/DedekindDomain/Ideal/Lemmas.lean,Mathlib/RingTheory/DedekindDomain/IntegralClosure.lean,Mathlib/RingTheory/FractionalIdeal/Extended.lean,Mathlib/RingTheory/Ideal/GoingUp.lean,Mathlib/RingTheory/Ideal/Maps.lean,Mathlib/RingTheory/Ideal/Norm/RelNorm.lean,Mathlib/RingTheory/Ideal/Operations.lean,Mathlib/RingTheory/Ideal/Over.lean,Mathlib/RingTheory/IntegralClosure/IntegralRestrict.lean,Mathlib/RingTheory/Localization/AtPrime/Basic.lean,Mathlib/RingTheory/Localization/AtPrime/Extension.lean,Mathlib/RingTheory/Localization/Basic.lean,Mathlib/RingTheory/Localization/FractionRing.lean,Mathlib/RingTheory/Trace/Basic.lean,Mathlib/RingTheory/Trace/Quotient.lean,Mathlib/Sandbox.lean,Mathlib/relNorm.lean |
38 |
n/a |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-merge-conflict-bot'] |
nobody |
0-59525 16 hours ago |
unknown |
unknown |
29544 |
sgouezel author:sgouezel |
class_abbrev branch. Just for bench |
Don't review, don't merge, please
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict |
1046/689 |
.github/actionlint.yml,.github/workflows/nightly-docgen.yml,.github/workflows/nightly_detect_failure.yml,.github/workflows/report-grind-regressions.yml,Cache/Requests.lean,Mathlib.lean,Mathlib/Algebra/Field/Rat.lean,Mathlib/Algebra/Homology/ExactSequence.lean,Mathlib/Algebra/Order/Ring/Rat.lean,Mathlib/Algebra/Order/Ring/Unbundled/Rat.lean,Mathlib/Algebra/Polynomial/Bivariate.lean,Mathlib/Algebra/Polynomial/Eval/Defs.lean,Mathlib/Algebra/Polynomial/Eval/SMul.lean,Mathlib/Algebra/Ring/Rat.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Instances.lean,Mathlib/Analysis/SpecialFunctions/Log/Summable.lean,Mathlib/CategoryTheory/Monoidal/Braided/Basic.lean,Mathlib/Computability/TMToPartrec.lean,Mathlib/Data/DFinsupp/Notation.lean,Mathlib/Data/FP/Basic.lean,Mathlib/Data/Finsupp/Notation.lean,Mathlib/Data/Int/Bitwise.lean,Mathlib/Data/Int/GCD.lean,Mathlib/Data/NNRat/Defs.lean,Mathlib/Data/Nat/GCD/Basic.lean,Mathlib/Data/Nat/GCD/BigOperators.lean,Mathlib/Data/Nat/PartENat.lean,Mathlib/Data/Nat/Prime/Defs.lean,Mathlib/Data/Rat/Cast/Defs.lean,Mathlib/Data/Rat/Defs.lean,Mathlib/Data/Rat/Floor.lean,Mathlib/Data/Rat/Lemmas.lean,Mathlib/Data/Seq/Basic.lean,Mathlib/Data/UInt.lean,Mathlib/Dynamics/PeriodicPts/Defs.lean,Mathlib/GroupTheory/Perm/Centralizer.lean,Mathlib/Init.lean,Mathlib/Lean/Expr/Rat.lean,Mathlib/Lean/Meta/CongrTheorems.lean,Mathlib/LinearAlgebra/PID.lean,Mathlib/LinearAlgebra/Quotient/Basic.lean,Mathlib/LinearAlgebra/Vandermonde.lean,Mathlib/Logic/Equiv/Prod.lean,Mathlib/NumberTheory/Ostrowski.lean,Mathlib/NumberTheory/Padics/PadicVal/Basic.lean,Mathlib/Order/Defs/LinearOrder.lean,Mathlib/Order/Defs/PartialOrder.lean,Mathlib/Order/Disjoint.lean,Mathlib/Order/Filter/Defs.lean,Mathlib/Probability/Distributions/Pareto.lean,Mathlib/RingTheory/Multiplicity.lean,Mathlib/Tactic.lean,Mathlib/Tactic/CategoryTheory/Reassoc.lean,Mathlib/Tactic/CategoryTheory/Refs.lean,Mathlib/Tactic/DeriveFintype.lean,Mathlib/Tactic/FieldSimp.lean,Mathlib/Tactic/Hint.lean,Mathlib/Tactic/Linarith/Oracle/SimplexAlgorithm/Datatypes.lean,Mathlib/Tactic/Linter/DeprecatedModule.lean,Mathlib/Tactic/Linter/Header.lean,Mathlib/Tactic/Linter/Lint.lean,Mathlib/Tactic/Linter/Style.lean,Mathlib/Tactic/NormNum/GCD.lean,Mathlib/Tactic/StacksAttribute.lean,Mathlib/Tactic/SuppressCompilation.lean,Mathlib/Tactic/ToAdditive/Frontend.lean,Mathlib/Tactic/WLOG.lean,Mathlib/Testing/Plausible/Sampleable.lean,Mathlib/Util/Notation3.lean,Mathlib/Util/ParseCommand.lean,Mathlib/Util/Superscript.lean,MathlibTest/AssertExists.lean,MathlibTest/CalcQuestionMark.lean,MathlibTest/Change.lean,MathlibTest/DeprecateTo.lean,MathlibTest/FieldSimp.lean,MathlibTest/FindSyntax.lean,MathlibTest/LibrarySearch/basic.lean,MathlibTest/LibrarySearch/mathlib.lean,MathlibTest/LibrarySearch/observe.lean,MathlibTest/MinImports.lean,MathlibTest/RewriteSearch/Basic.lean,MathlibTest/RewriteSearch/Polynomial.lean,MathlibTest/StacksAttribute.lean,MathlibTest/Subsingleton.lean,MathlibTest/Use.lean,MathlibTest/Variable.lean,MathlibTest/hint.lean,MathlibTest/lift.lean,MathlibTest/linarith.lean,MathlibTest/notation3.lean,MathlibTest/propose.lean,MathlibTest/renameBvar.lean,MathlibTest/rewrites.lean,MathlibTest/ring.lean,MathlibTest/says.lean,MathlibTest/success_if_fail_with_msg.lean,MathlibTest/toAdditive.lean,lake-manifest.json,lakefile.lean |
102 |
2 |
['sgouezel'] |
nobody |
0-55507 15 hours ago |
2-6588 2 days ago* |
0-0 0 seconds* |
22517 |
j-loreaux author:j-loreaux |
feat: `ℕ+` powers in semigroups |
---
[](https://gitpod.io/from-referrer/)
|
large-import
merge-conflict
WIP
|
275/28 |
Mathlib.lean,Mathlib/Algebra/Group/Defs.lean,Mathlib/Algebra/Group/Ext.lean,Mathlib/Algebra/Group/PNatPowAssoc.lean,Mathlib/Algebra/Group/PPow.lean,Mathlib/Algebra/Group/TypeTags/Basic.lean,Mathlib/Algebra/Ring/Ext.lean,Mathlib/Algebra/Ring/ULift.lean,Mathlib/Data/Num/Lemmas.lean,Mathlib/Data/Real/Basic.lean,Mathlib/Data/ZMod/Defs.lean,Mathlib/LinearAlgebra/LinearPMap.lean,Mathlib/NumberTheory/Dioph.lean,Mathlib/Tactic/ToAdditive/Frontend.lean |
14 |
6 |
['eric-wieser', 'github-actions', 'j-loreaux', 'leanprover-bot', 'mattrobball'] |
nobody |
0-47272 13 hours ago |
183-12482 5 months ago |
0-27 27 seconds |
26857 |
Thmoas-Guan author:Thmoas-Guan |
feat(Algebra): define associated graded structure for abelian group |
In this PR we define the associated graded structure for abelian group when given a filtration and only give some basic lemmas about it.
Further results would be given in #26858
---
[](https://gitpod.io/from-referrer/)
migrated from #22631
|
t-algebra
merge-conflict
awaiting-author
label:t-algebra$ |
153/0 |
Mathlib.lean,Mathlib/RingTheory/FilteredAlgebra/AssociatedGraded.lean |
2 |
12 |
['Thmoas-Guan', 'chrisflav', 'github-actions', 'mathlib4-merge-conflict-bot'] |
chrisflav assignee:chrisflav |
0-26592 7 hours ago |
0-26593 7 hours ago |
18-81638 18 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-ring-theory
merge-conflict
|
266/3 |
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/Ideal/Quotient/Basic.lean,Mathlib/RingTheory/TensorProduct/MvPolynomial.lean |
9 |
13 |
['chrisflav', 'erdOne', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
Vierkantor assignee:Vierkantor |
0-25069 6 hours ago |
0-25069 6 hours ago |
95-70661 95 days |
27320 |
Jlh18 author:Jlh18 |
doc (CategoryTheory/Bicategory/Grothendieck): rename Grothendieck to coGrothendieck |
Rename `CategoryTheory.Pseudofunctor.Grothendieck` to `CategoryTheory.Pseudofunctor.coGrothendieck`. Currently there are two inconsistent conventions taken in [`CategoryTheory.Grothendieck`](https://leanprover-community.github.io/mathlib4_docs/Mathlib/CategoryTheory/Grothendieck.html#CategoryTheory.Grothendieck) and [`CategoryTheory.Pseudofunctor.Grothendieck`](https://leanprover-community.github.io/mathlib4_docs/Mathlib/CategoryTheory/Bicategory/Grothendieck.html#CategoryTheory.Pseudofunctor.Grothendieck), namely the latter includes an `op` on the indexing category / base category of the Grothendieck construction.
Later on, I will make more PRs to introduce the version of `CategoryTheory.Pseudofunctor.Grothendieck` that does not have an `op`.
Zulip discussion: [#mathlib4 > Refactor Grothendieck from Pseudofunctor.Grothendieck](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Refactor.20Grothendieck.20from.20Pseudofunctor.2EGrothendieck/with/529165679).
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-category-theory
merge-conflict
|
45/37 |
Mathlib/CategoryTheory/Bicategory/Grothendieck.lean,Mathlib/CategoryTheory/FiberedCategory/Grothendieck.lean |
2 |
8 |
['Jlh18', 'github-actions', 'joelriou', 'kckennylau', 'mathlib4-merge-conflict-bot'] |
b-mehta assignee:b-mehta |
0-24722 6 hours ago |
0-24722 6 hours ago |
33-58465 33 days |
27933 |
grunweg author:grunweg |
chore(OrdNode): format code example in code blocks |
Wrap them in code blocks (and unindent them; that indentation is not needed any more).
This also avoids warnings from the linter in #27898.
-------
[](https://gitpod.io/from-referrer/)
|
t-data
merge-conflict
|
459/212 |
Mathlib/Data/Ordmap/Ordnode.lean |
1 |
4 |
['eric-wieser', 'github-actions', 'grunweg', 'mathlib4-merge-conflict-bot'] |
nobody |
0-24598 6 hours ago |
0-24599 6 hours ago |
39-69478 39 days |
28406 |
YaelDillies author:YaelDillies |
chore: rename `Mon_Class` to `MonObj` |
and `Comon_Class` to `ComonObj`.
`Grp_Class`, `CommGrp_Class` and `Mod_Class` will follow.
[Zulip](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Removing.20underscores.20from.20docs.23Mon_.2C.20docs.23Grp_.20.2E.2E.2E)
---
I will add the deprecations once we have agreed on the new names.
[](https://gitpod.io/from-referrer/)
|
t-category-theory
merge-conflict
|
315/268 |
Mathlib/Algebra/Category/CoalgCat/ComonEquivalence.lean,Mathlib/Algebra/Category/CommBialgCat.lean,Mathlib/Algebra/Category/Grp/LeftExactFunctor.lean,Mathlib/CategoryTheory/Bicategory/Monad/Basic.lean,Mathlib/CategoryTheory/Monad/EquivMon.lean,Mathlib/CategoryTheory/Monoidal/Bimod.lean,Mathlib/CategoryTheory/Monoidal/Bimon_.lean,Mathlib/CategoryTheory/Monoidal/Cartesian/CommGrp_.lean,Mathlib/CategoryTheory/Monoidal/Cartesian/CommMon_.lean,Mathlib/CategoryTheory/Monoidal/Cartesian/Comon_.lean,Mathlib/CategoryTheory/Monoidal/Cartesian/Grp_.lean,Mathlib/CategoryTheory/Monoidal/Cartesian/Mod_.lean,Mathlib/CategoryTheory/Monoidal/Cartesian/Mon_.lean,Mathlib/CategoryTheory/Monoidal/CommGrp_.lean,Mathlib/CategoryTheory/Monoidal/CommMon_.lean,Mathlib/CategoryTheory/Monoidal/Comon_.lean,Mathlib/CategoryTheory/Monoidal/Conv.lean,Mathlib/CategoryTheory/Monoidal/Grp_.lean,Mathlib/CategoryTheory/Monoidal/Hopf_.lean,Mathlib/CategoryTheory/Monoidal/Internal/FunctorCategory.lean,Mathlib/CategoryTheory/Monoidal/Internal/Module.lean,Mathlib/CategoryTheory/Monoidal/Internal/Types/Basic.lean,Mathlib/CategoryTheory/Monoidal/Internal/Types/CommGrp_.lean,Mathlib/CategoryTheory/Monoidal/Internal/Types/Grp_.lean,Mathlib/CategoryTheory/Monoidal/Mod_.lean,Mathlib/CategoryTheory/Monoidal/Mon_.lean,Mathlib/CategoryTheory/Monoidal/Opposite/Mon_.lean,Mathlib/CategoryTheory/Preadditive/CommGrp_.lean,Mathlib/Tactic/Attr/Register.lean,MathlibTest/CategoryTheory/Monoidal/MonTauto.lean |
30 |
10 |
['YaelDillies', 'github-actions', 'joelriou', 'mathlib4-merge-conflict-bot'] |
TwoFX assignee:TwoFX |
0-24475 6 hours ago |
0-24476 6 hours ago |
27-82127 27 days |
28767 |
chrisflav author:chrisflav |
feat(RingTheory/Extension/Presentation): lemmas for computation of Jacobian |
---
- [ ] depends on: #28725
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
merge-conflict
|
619/551 |
Mathlib.lean,Mathlib/LinearAlgebra/Determinant.lean,Mathlib/LinearAlgebra/LinearIndependent/Defs.lean,Mathlib/LinearAlgebra/LinearIndependent/Lemmas.lean,Mathlib/RingTheory/Extension/Presentation/Submersive.lean,Mathlib/RingTheory/Smooth/StandardSmooth.lean |
6 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
0-24350 6 hours ago |
0-24351 6 hours ago |
0-5220 1 hour |
29237 |
harahu author:harahu |
doc: capitalize archimedean |
Adjectives derived from people's last names are usually capitalized in English.
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict |
337/336 |
Counterexamples/MapFloor.lean,Mathlib/Algebra/ContinuedFractions/Computation/ApproximationCorollaries.lean,Mathlib/Algebra/Order/Archimedean/Basic.lean,Mathlib/Algebra/Order/Archimedean/Class.lean,Mathlib/Algebra/Order/Archimedean/Hom.lean,Mathlib/Algebra/Order/Archimedean/Submonoid.lean,Mathlib/Algebra/Order/CompleteField.lean,Mathlib/Algebra/Order/Hom/Basic.lean,Mathlib/Algebra/Order/Module/Archimedean.lean,Mathlib/Algebra/Order/Nonneg/Floor.lean,Mathlib/Algebra/Order/Ring/Archimedean.lean,Mathlib/Algebra/Order/Ring/Basic.lean,Mathlib/Algebra/Order/Ring/IsNonarchimedean.lean,Mathlib/Analysis/Calculus/UniformLimitsDeriv.lean,Mathlib/Analysis/Normed/Algebra/Ultra.lean,Mathlib/Analysis/Normed/Field/Ultra.lean,Mathlib/Analysis/Normed/Group/Seminorm.lean,Mathlib/Analysis/Normed/Group/Ultra.lean,Mathlib/Analysis/Normed/Order/Hom/Basic.lean,Mathlib/Analysis/Normed/Order/Hom/Ultra.lean,Mathlib/Analysis/Normed/Ring/Ultra.lean,Mathlib/Analysis/Normed/Unbundled/FiniteExtension.lean,Mathlib/Analysis/Normed/Unbundled/InvariantExtension.lean,Mathlib/Analysis/Normed/Unbundled/SeminormFromBounded.lean,Mathlib/Analysis/Normed/Unbundled/SeminormFromConst.lean,Mathlib/Analysis/Normed/Unbundled/SmoothingSeminorm.lean,Mathlib/Analysis/Normed/Unbundled/SpectralNorm.lean,Mathlib/Analysis/SpecialFunctions/Gamma/Deligne.lean,Mathlib/Data/Int/SuccPred.lean,Mathlib/Data/NNReal/Defs.lean,Mathlib/Data/Nat/SuccPred.lean,Mathlib/Data/Real/Embedding.lean,Mathlib/GroupTheory/Archimedean.lean,Mathlib/GroupTheory/ArchimedeanDensely.lean,Mathlib/NumberTheory/FunctionField.lean,Mathlib/NumberTheory/LSeries/DirichletContinuation.lean,Mathlib/NumberTheory/NumberField/FinitePlaces.lean,Mathlib/NumberTheory/Ostrowski.lean,Mathlib/NumberTheory/Padics/Complex.lean,Mathlib/NumberTheory/Padics/MahlerBasis.lean,Mathlib/NumberTheory/Padics/PadicIntegers.lean,Mathlib/NumberTheory/Padics/PadicNorm.lean,Mathlib/NumberTheory/Padics/ValuativeRel.lean,Mathlib/Order/Filter/AtTopBot/Archimedean.lean,Mathlib/Order/Interval/Finset/Box.lean,Mathlib/Order/SuccPred/Archimedean.lean,Mathlib/Order/SuccPred/Basic.lean,Mathlib/Order/SuccPred/IntervalSucc.lean,Mathlib/Order/SuccPred/LinearLocallyFinite.lean,Mathlib/Order/SuccPred/Tree.lean,Mathlib/RingTheory/DedekindDomain/AdicValuation.lean,Mathlib/RingTheory/HahnSeries/Lex.lean,Mathlib/RingTheory/Valuation/Archimedean.lean,Mathlib/RingTheory/Valuation/Basic.lean,Mathlib/RingTheory/Valuation/ValuativeRel/Basic.lean,Mathlib/Topology/Algebra/InfiniteSum/Nonarchimedean.lean,Mathlib/Topology/Algebra/Nonarchimedean/AdicTopology.lean,Mathlib/Topology/Algebra/Nonarchimedean/Bases.lean,Mathlib/Topology/Algebra/Nonarchimedean/Basic.lean,Mathlib/Topology/Algebra/Nonarchimedean/Completion.lean,Mathlib/Topology/Algebra/Nonarchimedean/TotallyDisconnected.lean,Mathlib/Topology/Algebra/OpenSubgroup.lean,Mathlib/Topology/Algebra/Order/Archimedean.lean,Mathlib/Topology/Algebra/Valued/LocallyCompact.lean,Mathlib/Topology/Algebra/Valued/NormedValued.lean,Mathlib/Topology/Algebra/Valued/ValuationTopology.lean,Mathlib/Topology/Connected/Basic.lean,Mathlib/Topology/MetricSpace/BundledFun.lean,Mathlib/Topology/MetricSpace/Ultra/Basic.lean,Mathlib/Topology/MetricSpace/Ultra/Pi.lean,Mathlib/Topology/MetricSpace/Ultra/TotallySeparated.lean,Mathlib/Topology/UniformSpace/Ultra/Basic.lean,Mathlib/Topology/UniformSpace/Ultra/Completion.lean,Mathlib/Topology/UniformSpace/Ultra/Constructions.lean |
74 |
4 |
['euprunin', 'github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
0-23737 6 hours ago |
0-23738 6 hours ago |
9-33674 9 days |
29353 |
Vierkantor author:Vierkantor |
chore(RingTheory): process porting notes, part 2 |
This PR goes through all the remaining porting notes in the RingTheory folder and fixes the ones that have an obvious solution.
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
tech debt
merge-conflict
|
210/321 |
Mathlib/Algebra/Module/Equiv/Defs.lean,Mathlib/Algebra/Module/LocalizedModule/Basic.lean,Mathlib/Algebra/Module/LocalizedModule/Submodule.lean,Mathlib/Algebra/Polynomial/Laurent.lean,Mathlib/FieldTheory/RatFunc/Basic.lean,Mathlib/NumberTheory/Cyclotomic/Basic.lean,Mathlib/NumberTheory/NumberField/FractionalIdeal.lean,Mathlib/NumberTheory/Padics/PadicIntegers.lean,Mathlib/RingTheory/LaurentSeries.lean,Mathlib/RingTheory/LocalRing/ResidueField/Ideal.lean,Mathlib/RingTheory/Localization/Algebra.lean,Mathlib/RingTheory/Localization/AtPrime/Basic.lean,Mathlib/RingTheory/Localization/Away/AdjoinRoot.lean,Mathlib/RingTheory/Localization/Away/Basic.lean,Mathlib/RingTheory/Localization/Basic.lean,Mathlib/RingTheory/Localization/Defs.lean,Mathlib/RingTheory/Localization/FractionRing.lean,Mathlib/RingTheory/Localization/Ideal.lean,Mathlib/RingTheory/Localization/Integral.lean,Mathlib/RingTheory/Localization/InvSubmonoid.lean,Mathlib/RingTheory/Localization/LocalizationLocalization.lean,Mathlib/RingTheory/Localization/NumDen.lean,Mathlib/RingTheory/Localization/Pi.lean,Mathlib/RingTheory/MatrixAlgebra.lean,Mathlib/RingTheory/Multiplicity.lean,Mathlib/RingTheory/MvPolynomial/Tower.lean,Mathlib/RingTheory/MvPowerSeries/Basic.lean,Mathlib/RingTheory/Noetherian/Defs.lean,Mathlib/RingTheory/NonUnitalSubsemiring/Basic.lean,Mathlib/RingTheory/Nullstellensatz.lean,Mathlib/RingTheory/Polynomial/Bernstein.lean,Mathlib/RingTheory/Polynomial/Content.lean,Mathlib/RingTheory/Polynomial/Cyclotomic/Roots.lean,Mathlib/RingTheory/Polynomial/Dickson.lean,Mathlib/RingTheory/Polynomial/Eisenstein/Basic.lean,Mathlib/RingTheory/Polynomial/GaussLemma.lean,Mathlib/RingTheory/Polynomial/Hermite/Basic.lean,Mathlib/RingTheory/Polynomial/Hermite/Gaussian.lean,Mathlib/RingTheory/Polynomial/RationalRoot.lean,Mathlib/RingTheory/PowerSeries/Basic.lean,Mathlib/RingTheory/ReesAlgebra.lean,Mathlib/RingTheory/RingHomProperties.lean,Mathlib/RingTheory/RingInvo.lean,Mathlib/RingTheory/RootsOfUnity/Basic.lean,Mathlib/RingTheory/RootsOfUnity/Minpoly.lean,Mathlib/RingTheory/SimpleModule/Basic.lean,Mathlib/RingTheory/Smooth/Basic.lean,Mathlib/RingTheory/Smooth/StandardSmooth.lean,Mathlib/RingTheory/Spectrum/Prime/Basic.lean,Mathlib/RingTheory/TensorProduct/Free.lean,Mathlib/RingTheory/Trace/Basic.lean,Mathlib/RingTheory/Unramified/Basic.lean,Mathlib/RingTheory/Valuation/Basic.lean,Mathlib/RingTheory/Valuation/Quotient.lean,Mathlib/RingTheory/Valuation/ValuationRing.lean,Mathlib/RingTheory/Valuation/ValuationSubring.lean,Mathlib/RingTheory/WittVector/Basic.lean,Mathlib/RingTheory/WittVector/Frobenius.lean,Mathlib/RingTheory/WittVector/Identities.lean,Mathlib/RingTheory/WittVector/IsPoly.lean,Mathlib/RingTheory/WittVector/MulCoeff.lean |
61 |
4 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
0-23614 6 hours ago |
0-23614 6 hours ago |
7-725 7 days |
29596 |
alreadydone author:alreadydone |
chore(Algebra): extract `Submonoid.IsLocalizationMap` |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
label:t-algebra$ |
268/115 |
Mathlib.lean,Mathlib/Algebra/Module/LocalizedModule/IsLocalization.lean,Mathlib/GroupTheory/MonoidLocalization/Basic.lean,Mathlib/GroupTheory/MonoidLocalization/Lemmas.lean,Mathlib/GroupTheory/MonoidLocalization/MonoidWithZero.lean,Mathlib/RingTheory/Localization/Basic.lean,Mathlib/RingTheory/Localization/Defs.lean,Mathlib/RingTheory/Smooth/StandardSmooth.lean |
8 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
0-23369 6 hours ago |
0-23370 6 hours ago |
0-42377 11 hours |
29581 |
sgouezel author:sgouezel |
Sg test3 |
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict
WIP
|
2707/3264 |
.github/actionlint.yml,.github/workflows/nightly-docgen.yml,.github/workflows/nightly_detect_failure.yml,.github/workflows/report-grind-regressions.yml,Cache/Requests.lean,Mathlib.lean,Mathlib/Algebra/Algebra/RestrictScalars.lean,Mathlib/Algebra/Algebra/Subalgebra/Basic.lean,Mathlib/Algebra/Field/Rat.lean,Mathlib/Algebra/Homology/ExactSequence.lean,Mathlib/Algebra/Order/Ring/Rat.lean,Mathlib/Algebra/Order/Ring/Unbundled/Rat.lean,Mathlib/Algebra/Polynomial/Bivariate.lean,Mathlib/Algebra/Polynomial/Eval/Defs.lean,Mathlib/Algebra/Polynomial/Eval/SMul.lean,Mathlib/Algebra/Ring/InjSurj.lean,Mathlib/Algebra/Ring/Rat.lean,Mathlib/Algebra/Ring/Subring/Defs.lean,Mathlib/Analysis/Analytic/Composition.lean,Mathlib/Analysis/Analytic/Order.lean,Mathlib/Analysis/CStarAlgebra/ApproximateUnit.lean,Mathlib/Analysis/CStarAlgebra/Basic.lean,Mathlib/Analysis/CStarAlgebra/CStarMatrix.lean,Mathlib/Analysis/CStarAlgebra/Classes.lean,Mathlib/Analysis/CStarAlgebra/CompletelyPositiveMap.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Basic.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Instances.lean,Mathlib/Analysis/CStarAlgebra/Matrix.lean,Mathlib/Analysis/CStarAlgebra/Module/Constructions.lean,Mathlib/Analysis/CStarAlgebra/Module/Defs.lean,Mathlib/Analysis/CStarAlgebra/Multiplier.lean,Mathlib/Analysis/CStarAlgebra/Unitization.lean,Mathlib/Analysis/CStarAlgebra/lpSpace.lean,Mathlib/Analysis/Calculus/BumpFunction/FiniteDimension.lean,Mathlib/Analysis/Calculus/ContDiff/Basic.lean,Mathlib/Analysis/Calculus/ContDiff/Operations.lean,Mathlib/Analysis/Calculus/DSlope.lean,Mathlib/Analysis/Calculus/Deriv/CompMul.lean,Mathlib/Analysis/Calculus/Deriv/Inv.lean,Mathlib/Analysis/Calculus/DiffContOnCl.lean,Mathlib/Analysis/Calculus/FDeriv/Equiv.lean,Mathlib/Analysis/Calculus/FDeriv/Mul.lean,Mathlib/Analysis/Calculus/FDeriv/Symmetric.lean,Mathlib/Analysis/Calculus/LineDeriv/QuadraticMap.lean,Mathlib/Analysis/Calculus/MeanValue.lean,Mathlib/Analysis/Calculus/SmoothSeries.lean,Mathlib/Analysis/Calculus/UniformLimitsDeriv.lean,Mathlib/Analysis/Complex/Basic.lean,Mathlib/Analysis/Complex/Hadamard.lean,Mathlib/Analysis/Complex/Norm.lean,Mathlib/Analysis/Complex/Tietze.lean,Mathlib/Analysis/Fourier/FourierTransform.lean,Mathlib/Analysis/Fourier/FourierTransformDeriv.lean,Mathlib/Analysis/InnerProductSpace/Basic.lean,Mathlib/Analysis/InnerProductSpace/Calculus.lean,Mathlib/Analysis/InnerProductSpace/Completion.lean,Mathlib/Analysis/InnerProductSpace/Defs.lean,Mathlib/Analysis/InnerProductSpace/MulOpposite.lean,Mathlib/Analysis/InnerProductSpace/OfNorm.lean,Mathlib/Analysis/InnerProductSpace/Orthonormal.lean,Mathlib/Analysis/InnerProductSpace/PiL2.lean,Mathlib/Analysis/InnerProductSpace/ProdL2.lean,Mathlib/Analysis/InnerProductSpace/Projection/Minimal.lean,Mathlib/Analysis/InnerProductSpace/Subspace.lean,Mathlib/Analysis/InnerProductSpace/l2Space.lean,Mathlib/Analysis/LocallyConvex/WithSeminorms.lean,Mathlib/Analysis/Matrix.lean,Mathlib/Analysis/Meromorphic/Basic.lean,Mathlib/Analysis/Normed/Affine/ContinuousAffineMap.lean,Mathlib/Analysis/Normed/Algebra/Spectrum.lean,Mathlib/Analysis/Normed/Algebra/TrivSqZeroExt.lean,Mathlib/Analysis/Normed/Algebra/Unitization.lean,Mathlib/Analysis/Normed/Algebra/UnitizationL1.lean,Mathlib/Analysis/Normed/Field/Basic.lean,Mathlib/Analysis/Normed/Field/WithAbs.lean,Mathlib/Analysis/Normed/Group/AddCircle.lean,Mathlib/Analysis/Normed/Group/Basic.lean,Mathlib/Analysis/Normed/Group/Completion.lean,Mathlib/Analysis/Normed/Group/Constructions.lean,Mathlib/Analysis/Normed/Group/Continuity.lean,Mathlib/Analysis/Normed/Group/Hom.lean,Mathlib/Analysis/Normed/Group/Int.lean,Mathlib/Analysis/Normed/Group/Quotient.lean,Mathlib/Analysis/Normed/Group/Rat.lean,Mathlib/Analysis/Normed/Group/SemiNormedGrp.lean,Mathlib/Analysis/Normed/Group/Subgroup.lean,Mathlib/Analysis/Normed/Group/Submodule.lean,Mathlib/Analysis/Normed/Group/Ultra.lean,Mathlib/Analysis/Normed/Group/Uniform.lean,Mathlib/Analysis/Normed/Lp/PiLp.lean,Mathlib/Analysis/Normed/Lp/ProdLp.lean,Mathlib/Analysis/Normed/Lp/lpSpace.lean,Mathlib/Analysis/Normed/Module/Basic.lean,Mathlib/Analysis/Normed/Module/Completion.lean,Mathlib/Analysis/Normed/Module/FiniteDimension.lean,Mathlib/Analysis/Normed/Operator/BoundedLinearMaps.lean,Mathlib/Analysis/Normed/Order/Hom/Basic.lean,Mathlib/Analysis/Normed/Order/Hom/Ultra.lean,Mathlib/Analysis/Normed/Ring/Basic.lean,Mathlib/Analysis/Normed/Ring/Lemmas.lean |
245 |
3 |
['leanprover-bot', 'mathlib4-merge-conflict-bot', 'sgouezel'] |
nobody |
0-2741 45 minutes ago |
1-11338 1 day ago* |
0-0 0 seconds* |
29614 |
sgouezel author:sgouezel |
Sg test4 |
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict |
2707/3264 |
.github/actionlint.yml,.github/workflows/nightly-docgen.yml,.github/workflows/nightly_detect_failure.yml,.github/workflows/report-grind-regressions.yml,Cache/Requests.lean,Mathlib.lean,Mathlib/Algebra/Algebra/RestrictScalars.lean,Mathlib/Algebra/Algebra/Subalgebra/Basic.lean,Mathlib/Algebra/Field/Rat.lean,Mathlib/Algebra/Homology/ExactSequence.lean,Mathlib/Algebra/Order/Ring/Rat.lean,Mathlib/Algebra/Order/Ring/Unbundled/Rat.lean,Mathlib/Algebra/Polynomial/Bivariate.lean,Mathlib/Algebra/Polynomial/Eval/Defs.lean,Mathlib/Algebra/Polynomial/Eval/SMul.lean,Mathlib/Algebra/Ring/InjSurj.lean,Mathlib/Algebra/Ring/Rat.lean,Mathlib/Algebra/Ring/Subring/Defs.lean,Mathlib/Analysis/Analytic/Composition.lean,Mathlib/Analysis/Analytic/Order.lean,Mathlib/Analysis/CStarAlgebra/ApproximateUnit.lean,Mathlib/Analysis/CStarAlgebra/Basic.lean,Mathlib/Analysis/CStarAlgebra/CStarMatrix.lean,Mathlib/Analysis/CStarAlgebra/Classes.lean,Mathlib/Analysis/CStarAlgebra/CompletelyPositiveMap.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Basic.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Instances.lean,Mathlib/Analysis/CStarAlgebra/Matrix.lean,Mathlib/Analysis/CStarAlgebra/Module/Constructions.lean,Mathlib/Analysis/CStarAlgebra/Module/Defs.lean,Mathlib/Analysis/CStarAlgebra/Multiplier.lean,Mathlib/Analysis/CStarAlgebra/Unitization.lean,Mathlib/Analysis/CStarAlgebra/lpSpace.lean,Mathlib/Analysis/Calculus/BumpFunction/FiniteDimension.lean,Mathlib/Analysis/Calculus/ContDiff/Basic.lean,Mathlib/Analysis/Calculus/ContDiff/Operations.lean,Mathlib/Analysis/Calculus/DSlope.lean,Mathlib/Analysis/Calculus/Deriv/CompMul.lean,Mathlib/Analysis/Calculus/Deriv/Inv.lean,Mathlib/Analysis/Calculus/DiffContOnCl.lean,Mathlib/Analysis/Calculus/FDeriv/Equiv.lean,Mathlib/Analysis/Calculus/FDeriv/Mul.lean,Mathlib/Analysis/Calculus/FDeriv/Symmetric.lean,Mathlib/Analysis/Calculus/LineDeriv/QuadraticMap.lean,Mathlib/Analysis/Calculus/MeanValue.lean,Mathlib/Analysis/Calculus/SmoothSeries.lean,Mathlib/Analysis/Calculus/UniformLimitsDeriv.lean,Mathlib/Analysis/Complex/Basic.lean,Mathlib/Analysis/Complex/Hadamard.lean,Mathlib/Analysis/Complex/Norm.lean,Mathlib/Analysis/Complex/Tietze.lean,Mathlib/Analysis/Fourier/FourierTransform.lean,Mathlib/Analysis/Fourier/FourierTransformDeriv.lean,Mathlib/Analysis/InnerProductSpace/Basic.lean,Mathlib/Analysis/InnerProductSpace/Calculus.lean,Mathlib/Analysis/InnerProductSpace/Completion.lean,Mathlib/Analysis/InnerProductSpace/Defs.lean,Mathlib/Analysis/InnerProductSpace/MulOpposite.lean,Mathlib/Analysis/InnerProductSpace/OfNorm.lean,Mathlib/Analysis/InnerProductSpace/Orthonormal.lean,Mathlib/Analysis/InnerProductSpace/PiL2.lean,Mathlib/Analysis/InnerProductSpace/ProdL2.lean,Mathlib/Analysis/InnerProductSpace/Projection/Minimal.lean,Mathlib/Analysis/InnerProductSpace/Subspace.lean,Mathlib/Analysis/InnerProductSpace/l2Space.lean,Mathlib/Analysis/LocallyConvex/WithSeminorms.lean,Mathlib/Analysis/Matrix.lean,Mathlib/Analysis/Meromorphic/Basic.lean,Mathlib/Analysis/Normed/Affine/ContinuousAffineMap.lean,Mathlib/Analysis/Normed/Algebra/Spectrum.lean,Mathlib/Analysis/Normed/Algebra/TrivSqZeroExt.lean,Mathlib/Analysis/Normed/Algebra/Unitization.lean,Mathlib/Analysis/Normed/Algebra/UnitizationL1.lean,Mathlib/Analysis/Normed/Field/Basic.lean,Mathlib/Analysis/Normed/Field/WithAbs.lean,Mathlib/Analysis/Normed/Group/AddCircle.lean,Mathlib/Analysis/Normed/Group/Basic.lean,Mathlib/Analysis/Normed/Group/Completion.lean,Mathlib/Analysis/Normed/Group/Constructions.lean,Mathlib/Analysis/Normed/Group/Continuity.lean,Mathlib/Analysis/Normed/Group/Hom.lean,Mathlib/Analysis/Normed/Group/Int.lean,Mathlib/Analysis/Normed/Group/Quotient.lean,Mathlib/Analysis/Normed/Group/Rat.lean,Mathlib/Analysis/Normed/Group/SemiNormedGrp.lean,Mathlib/Analysis/Normed/Group/Subgroup.lean,Mathlib/Analysis/Normed/Group/Submodule.lean,Mathlib/Analysis/Normed/Group/Ultra.lean,Mathlib/Analysis/Normed/Group/Uniform.lean,Mathlib/Analysis/Normed/Lp/PiLp.lean,Mathlib/Analysis/Normed/Lp/ProdLp.lean,Mathlib/Analysis/Normed/Lp/lpSpace.lean,Mathlib/Analysis/Normed/Module/Basic.lean,Mathlib/Analysis/Normed/Module/Completion.lean,Mathlib/Analysis/Normed/Module/FiniteDimension.lean,Mathlib/Analysis/Normed/Operator/BoundedLinearMaps.lean,Mathlib/Analysis/Normed/Order/Hom/Basic.lean,Mathlib/Analysis/Normed/Order/Hom/Ultra.lean,Mathlib/Analysis/Normed/Ring/Basic.lean,Mathlib/Analysis/Normed/Ring/Lemmas.lean |
245 |
0 |
[] |
nobody |
0-2715 45 minutes ago |
0-8670 2 hours ago* |
0-0 0 seconds* |
13158 |
erdOne author:erdOne |
refactor(RingTheory/OreLocalization/Module): remove `LocalizedModule.mk`. |
---
- [x] depends on: #13151
- [ ] depends on: #13156
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
blocked-by-other-PR
label:t-algebra$ |
49/48 |
Mathlib/RingTheory/OreLocalization/Basic.lean,Mathlib/RingTheory/OreLocalization/Module.lean |
2 |
1 |
['leanprover-community-mathlib4-bot'] |
nobody |
430-76019 1 year ago |
430-76042 1 year ago |
0-0 0 seconds |
14889 |
yuma-mizuno author:yuma-mizuno |
feat(CategoryTheory/Bicategory/Monad): define monad in bicategory |
---
- [ ] depends on: #12107
[](https://gitpod.io/from-referrer/)
|
t-category-theory
merge-conflict
blocked-by-other-PR
WIP
|
1566/12 |
Mathlib.lean,Mathlib/CategoryTheory/Bicategory/Functor/Oplax.lean,Mathlib/CategoryTheory/Bicategory/LocallyDiscrete.lean,Mathlib/CategoryTheory/Bicategory/Monad/Adjunction.lean,Mathlib/CategoryTheory/Bicategory/Monad/Basic.lean,Mathlib/CategoryTheory/Bicategory/Monad/Cat.lean,Mathlib/CategoryTheory/Monad/Basic.lean,Mathlib/Tactic.lean,Mathlib/Tactic/CategoryTheory/Coherence.lean,Mathlib/Tactic/Widget/StringDiagram.lean,scripts/noshake.json,test/StringDiagram.lean,widget/src/penrose/monoidal.dsl,widget/src/penrose/monoidal.sty |
14 |
2 |
['github-actions', 'leanprover-community-mathlib4-bot'] |
nobody |
409-8945 1 year ago |
421-20183 1 year ago |
0-0 0 seconds |
12879 |
grunweg author:grunweg |
feat: port ge_or_gt linter from mathlib3 |
Code works and is essentially green: next step is to split up into separate PRs.
Feedback welcome on whether:
- all the test changes are good, or I should simply allow it in more cases
- if calc blocks need to be explicitly exempt
---
- [ ] depends on: #12933
- [ ] depends on: #12934
- [ ] depends on: #12931
[](https://gitpod.io/from-referrer/)
|
tech debt
t-linter
merge-conflict
blocked-by-other-PR
|
736/319 |
Archive/Imo/Imo1960Q1.lean,Archive/Imo/Imo1962Q1.lean,Archive/Imo/Imo1988Q6.lean,Archive/Imo/Imo1994Q1.lean,Archive/Imo/Imo2001Q2.lean,Archive/Imo/Imo2005Q3.lean,Archive/Imo/Imo2006Q3.lean,Archive/Imo/Imo2008Q2.lean,Archive/Imo/Imo2008Q3.lean,Archive/Imo/Imo2008Q4.lean,Archive/Imo/Imo2011Q5.lean,Archive/Imo/Imo2019Q4.lean,Archive/Sensitivity.lean,Archive/Wiedijk100Theorems/AreaOfACircle.lean,Archive/Wiedijk100Theorems/BallotProblem.lean,Archive/Wiedijk100Theorems/BirthdayProblem.lean,Archive/Wiedijk100Theorems/CubingACube.lean,Mathlib.lean,Mathlib/Algebra/DualNumber.lean,Mathlib/Algebra/Order/CauSeq/BigOperators.lean,Mathlib/Algebra/Order/Field/Basic.lean,Mathlib/Algebra/Order/Ring/Defs.lean,Mathlib/Algebra/Polynomial/Basic.lean,Mathlib/Algebra/Polynomial/Degree/Definitions.lean,Mathlib/Algebra/Star/CHSH.lean,Mathlib/Analysis/Analytic/Basic.lean,Mathlib/Analysis/Calculus/UniformLimitsDeriv.lean,Mathlib/Analysis/Complex/Hadamard.lean,Mathlib/Analysis/Complex/UpperHalfPlane/Basic.lean,Mathlib/Analysis/InnerProductSpace/Projection.lean,Mathlib/Analysis/Normed/Group/ControlledClosure.lean,Mathlib/Analysis/NormedSpace/MStructure.lean,Mathlib/Analysis/SpecialFunctions/Log/Base.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Basic.lean,Mathlib/Combinatorics/SimpleGraph/DegreeSum.lean,Mathlib/Combinatorics/SimpleGraph/LapMatrix.lean,Mathlib/Computability/AkraBazzi/AkraBazzi.lean,Mathlib/Computability/AkraBazzi/GrowsPolynomially.lean,Mathlib/Data/Complex/Basic.lean,Mathlib/Data/FP/Basic.lean,Mathlib/Data/Finset/Basic.lean,Mathlib/Data/Finset/Fold.lean,Mathlib/Data/Finsupp/Notation.lean,Mathlib/Data/Int/Lemmas.lean,Mathlib/Data/Nat/Dist.lean,Mathlib/Data/Nat/Lattice.lean,Mathlib/Data/Nat/Parity.lean,Mathlib/Data/Nat/Upto.lean,Mathlib/Data/Ordmap/Ordset.lean,Mathlib/Data/PNat/Basic.lean,Mathlib/Data/UInt.lean,Mathlib/GroupTheory/Coxeter/Length.lean,Mathlib/MeasureTheory/Constructions/Polish.lean,Mathlib/MeasureTheory/Covering/Besicovitch.lean,Mathlib/MeasureTheory/Covering/Vitali.lean,Mathlib/MeasureTheory/Covering/VitaliFamily.lean,Mathlib/MeasureTheory/Integral/Layercake.lean,Mathlib/NumberTheory/LegendreSymbol/JacobiSymbol.lean,Mathlib/NumberTheory/Padics/Hensel.lean,Mathlib/NumberTheory/Padics/PadicNorm.lean,Mathlib/NumberTheory/PellMatiyasevic.lean,Mathlib/NumberTheory/Rayleigh.lean,Mathlib/Order/Filter/AtTopBot.lean,Mathlib/Probability/Process/Stopping.lean,Mathlib/RingTheory/Adjoin/Basic.lean,Mathlib/RingTheory/Polynomial/Basic.lean,Mathlib/SetTheory/Ordinal/Notation.lean,Mathlib/Tactic.lean,Mathlib/Tactic/CancelDenoms/Core.lean,Mathlib/Tactic/Common.lean,Mathlib/Tactic/IntervalCases.lean,Mathlib/Tactic/Linarith/Datatypes.lean,Mathlib/Tactic/Linarith/Lemmas.lean,Mathlib/Tactic/Linarith/Oracle/FourierMotzkin.lean,Mathlib/Tactic/Linter/GeOrGt.lean,Mathlib/Tactic/Linter/Style.lean,Mathlib/Tactic/NormNum/GCD.lean,Mathlib/Tactic/NormNum/Inv.lean,Mathlib/Tactic/Ring/Basic.lean,Mathlib/Topology/Category/Profinite/Nobeling.lean,Mathlib/Topology/ContinuousFunction/Bounded.lean,Mathlib/Topology/MetricSpace/CauSeqFilter.lean,Mathlib/Topology/MetricSpace/Cauchy.lean,Mathlib/Topology/MetricSpace/Closeds.lean,Mathlib/Topology/Sequences.lean,scripts/lint-style.py,test/Explode.lean,test/GCongr/inequalities.lean,test/GeOrGt.lean,test/LibrarySearch/IsCompact.lean,test/LibrarySearch/basic.lean,test/Recall.lean,test/Rify.lean,test/Use.lean,test/cancel_denoms.lean,test/congr.lean,test/delabLinearIndependent.lean,test/delaborators.lean,test/interval_cases.lean,test/linarith.lean |
109 |
3 |
['github-actions', 'grunweg', 'leanprover-community-mathlib4-bot'] |
nobody |
409-8942 1 year ago |
430-76042 1 year ago |
0-15202 4 hours |
13057 |
alreadydone author:alreadydone |
feat(NumberTheory): characterize elliptic divisibility sequences |
Main results:
+ Every `normEDS` is an elliptic divisibility sequence (EDS). The key proof is `rel₄_of_anti_oddRec_evenRec`, based on my original argument first published on [MathSE](https://math.stackexchange.com/a/4903422/12932)
+ Conversely, every EDS is equal to some `normEDS` (assuming that the first two terms are not zero divisors)
---
- [ ] depends on: #13155
- [x] depends on: #13153
- [x] depends on: #10843
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-number-theory
merge-conflict
blocked-by-other-PR
label:t-algebra$ |
1032/55 |
Mathlib/Algebra/Ring/NegOnePow.lean,Mathlib/Data/Int/Defs.lean,Mathlib/Data/Int/Parity.lean,Mathlib/GroupTheory/Perm/Sign.lean,Mathlib/NumberTheory/EllipticDivisibilitySequence.lean |
5 |
6 |
['Multramate', 'alreadydone', 'kbuzzard', 'leanprover-community-mathlib4-bot'] |
nobody |
409-8942 1 year ago |
459-50330 1 year ago |
0-34665 9 hours |
10842 |
mcdoll author:mcdoll |
chore: simplify proofs using new positivity extensions and tests |
---
- [x] depends on: #10661
- [ ] depends on: #10796
[](https://gitpod.io/from-referrer/)
|
merge-conflict
blocked-by-other-PR
WIP
|
98/50 |
Mathlib/Analysis/Convolution.lean,Mathlib/Analysis/SpecialFunctions/Gaussian.lean,Mathlib/MeasureTheory/Covering/Differentiation.lean,Mathlib/MeasureTheory/Function/ConditionalExpectation/CondexpL1.lean,Mathlib/MeasureTheory/Function/ConditionalExpectation/Real.lean,Mathlib/MeasureTheory/Function/ConditionalExpectation/Unique.lean,Mathlib/MeasureTheory/Function/ContinuousMapDense.lean,Mathlib/MeasureTheory/Integral/Bochner.lean,Mathlib/MeasureTheory/Measure/Tilted.lean,Mathlib/Probability/Martingale/Upcrossing.lean,Mathlib/Probability/Moments.lean,Mathlib/Probability/Variance.lean,Mathlib/Tactic/Positivity/Core.lean,test/positivity.lean |
14 |
1 |
['leanprover-community-mathlib4-bot'] |
nobody |
409-8940 1 year ago |
473-12161 1 year ago |
0-0 0 seconds |
7564 |
shuxuezhuyi author:shuxuezhuyi |
feat(Topology/Algebra/Order): extend strictly monotone function on `Ioo` to homeomorphism on `Icc` |
A strictly monotone function between open intervals can be extended to a homeomorphism between the closed intervals.
---
- [ ] depends on: #7351
[](https://gitpod.io/from-referrer/)
|
t-topology
merge-conflict
blocked-by-other-PR
|
162/0 |
Mathlib.lean,Mathlib/Topology/Algebra/Order/IccExtendFromIoo.lean |
2 |
1 |
['leanprover-community-mathlib4-bot'] |
nobody |
409-8938 1 year ago |
430-76042 1 year ago |
0-0 0 seconds |
8364 |
thorimur author:thorimur |
feat: `refine?` |
This PR adds `refine? e`, which suggests replacing unsynthesized `_`'s in `e` with `?_` in order to make `refine e'` work:
```lean
example : Nat → Nat := by
refine? fun (_ : _) => _ -- Try this: refine fun (_ : _) => ?_
```
Note that this only suggests replacements for `_`'s present in the syntax; to create goals for implicit or instance arguments, the user is expected to use `refine'`.
---
I'm especially open to suggestions on the filename (currently `RefineFix`).
I'm also curious if this behaves as expected! Feel free to try it out "in real life" and comment here on edge cases.
- [ ] depends on: #8503
[](https://gitpod.io/from-referrer/)
|
t-meta
merge-conflict
blocked-by-other-PR
|
684/5 |
Mathlib.lean,Mathlib/Lean/CoreM.lean,Mathlib/Lean/Elab/Tactic/ElabTerm.lean,Mathlib/Lean/Elab/Term.lean,Mathlib/Tactic.lean,Mathlib/Tactic/RefineFix.lean,Mathlib/Util/Delaborators.lean,Mathlib/Util/Syntax.lean,test/RefineFix.lean |
9 |
5 |
['j-loreaux', 'leanprover-community-mathlib4-bot', 'thorimur'] |
nobody |
409-8938 1 year ago |
430-76042 1 year ago |
6-59794 6 days |
7512 |
Komyyy author:Komyyy |
perf: override the data structures of coinductive types |
The data structures of the model of coinductive types (`Stream'`, `Computation`, `Stream'.Seq`) are inefficient, so we override their data structures.
---
- [x] depends on: #7514
- [ ] depends on: leanprover/lean4#2292
- [x] depends on: leanprover/std4#371
- [x] depends on: #8460
[](https://gitpod.io/from-referrer/)
|
t-meta
merge-conflict
blocked-by-core-PR
blocked-by-other-PR
WIP
|
6919/3700 |
Mathlib.lean,Mathlib/Algebra/ContinuedFractions/Basic.lean,Mathlib/Algebra/ContinuedFractions/Computation/ApproximationCorollaries.lean,Mathlib/Algebra/ContinuedFractions/Computation/Approximations.lean,Mathlib/Algebra/ContinuedFractions/Computation/Basic.lean,Mathlib/Algebra/ContinuedFractions/Computation/CorrectnessTerminating.lean,Mathlib/Algebra/ContinuedFractions/Computation/TerminatesIffRat.lean,Mathlib/Algebra/ContinuedFractions/Computation/Translations.lean,Mathlib/Algebra/ContinuedFractions/ContinuantRecurrence.lean,Mathlib/Algebra/ContinuedFractions/EvalEquiv.lean,Mathlib/Algebra/ContinuedFractions/Real.lean,Mathlib/Algebra/ContinuedFractions/TerminatedStable.lean,Mathlib/Algebra/ContinuedFractions/Translations.lean,Mathlib/Combinatorics/Hindman.lean,Mathlib/Control/Fix.lean,Mathlib/Control/LawfulFix.lean,Mathlib/Data/Seq/Computation.lean,Mathlib/Data/Seq/Parallel.lean,Mathlib/Data/Seq/Seq.lean,Mathlib/Data/Seq/WSeq.lean,Mathlib/Data/Stream.lean,lean-toolchain |
22 |
2 |
['digama0', 'leanprover-community-mathlib4-bot'] |
nobody |
409-8938 1 year ago |
470-72979 1 year ago |
0-0 0 seconds |
4785 |
thorimur author:thorimur |
feat: ExprWithLevels |
This introduces `ExprWithLevels`, a means of emulating universe polymorphism for non-constants during metaprogramming. [Description pending]
- [ ] depends on: #4786
---
[](https://gitpod.io/from-referrer/)
|
t-meta
merge-conflict
blocked-by-other-PR
|
491/1 |
Mathlib.lean,Mathlib/Lean/Meta/AppBuilder.lean,Mathlib/Lean/Meta/Basic.lean,Mathlib/Lean/Meta/ExprWithLevels.lean |
4 |
1 |
['kim-em'] |
nobody |
409-8937 1 year ago |
473-12161 1 year ago |
0-0 0 seconds |
13852 |
FR-vdash-bot author:FR-vdash-bot |
perf: skip some typeclasses in TC search |
---
- [ ] depends on: #7873
[](https://gitpod.io/from-referrer/)
|
slow-typeclass-synthesis
merge-conflict
blocked-by-other-PR
|
45/33 |
Mathlib/Algebra/Group/Defs.lean,Mathlib/Algebra/Ring/Defs.lean,Mathlib/RingTheory/Norm.lean |
3 |
21 |
['FR-vdash-bot', 'MichaelStollBayreuth', 'github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot'] |
nobody |
404-65326 1 year ago |
404-65327 1 year ago |
0-0 0 seconds |
7565 |
shuxuezhuyi author:shuxuezhuyi |
feat(Topology/Algebra/Order): extend homeomorphism of `Ioo` to `Icc` |
We extend the homeomorphisms between open intervals to homeomorphisms between the closed intervals.
---
- [ ] depends on: #7018
- [ ] depends on: #7351
- [ ] depends on: #7564
[](https://gitpod.io/from-referrer/)
|
t-order
t-topology
merge-conflict
blocked-by-other-PR
|
389/5 |
Mathlib.lean,Mathlib/Data/Set/Intervals/Image.lean,Mathlib/Order/Directed.lean,Mathlib/Topology/Algebra/Order/IccExtendFromIoo.lean,Mathlib/Topology/Algebra/Order/IntermediateValue.lean |
5 |
1 |
['leanprover-community-mathlib4-bot'] |
nobody |
395-2591 1 year ago |
395-2591 1 year ago |
0-0 0 seconds |
11520 |
thorimur author:thorimur |
feat: `linting_rules` and deprecated syntax |
---
Experimental. WIP. Might not be performance-viable.
- [ ] depends on: #11519
[](https://gitpod.io/from-referrer/)
|
t-meta
merge-conflict
blocked-by-other-PR
|
1016/0 |
Mathlib.lean,Mathlib/Command/Linter.lean,Mathlib/Command/Linter/Deprecated.lean,Mathlib/Command/Linter/LintingRules.lean,Mathlib/Command/SyntaxRules.lean,Mathlib/Command/SyntaxRules/Attr.lean,Mathlib/Command/SyntaxRules/Elab.lean,Mathlib/Command/SyntaxRules/Header.lean,Mathlib/Command/SyntaxRules/Util.lean,Mathlib/Tactic/Common.lean,scripts/noshake.json |
11 |
11 |
['leanprover-bot', 'leanprover-community-mathlib4-bot', 'thorimur'] |
nobody |
393-85196 1 year ago |
393-85196 1 year ago |
0-0 0 seconds |
9154 |
FR-vdash-bot author:FR-vdash-bot |
feat: `npow` / `nsmul` / `Nat.cast`/ `zpow` / `zsmul` implemented using `Nat.binaryRec` |
---
- [ ] depends on: https://github.com/leanprover/lean4/pull/3756
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
awaiting-author
blocked-by-other-PR
label:t-algebra$ |
168/359 |
Mathlib/Algebra/Group/Defs.lean,Mathlib/Computability/PartrecCode.lean,Mathlib/Computability/Primrec.lean,Mathlib/Data/Bool/Basic.lean,Mathlib/Data/Int/Bitwise.lean,Mathlib/Data/Nat/Bits.lean,Mathlib/Data/Nat/Bitwise.lean,Mathlib/Data/Nat/Digits.lean,Mathlib/Data/Nat/EvenOddRec.lean,Mathlib/Data/Nat/Fib/Basic.lean,Mathlib/Data/Nat/Multiplicity.lean,Mathlib/Data/Nat/Order/Basic.lean,Mathlib/Data/Nat/Parity.lean,Mathlib/Data/Nat/Size.lean,Mathlib/Data/Num/Lemmas.lean,Mathlib/Init/Data/Nat/Bitwise.lean,Mathlib/LinearAlgebra/TensorProduct/Graded/Internal.lean,Mathlib/Logic/Basic.lean,Mathlib/Logic/Denumerable.lean,Mathlib/Logic/Encodable/Basic.lean,Mathlib/Logic/Equiv/Basic.lean,Mathlib/Logic/Equiv/Nat.lean,lake-manifest.json,lakefile.lean,test/zmod.lean |
25 |
7 |
['FR-vdash-bot', 'eric-wieser', 'kim-em', 'leanprover-community-mathlib4-bot'] |
nobody |
393-84669 1 year ago |
393-84669 1 year ago |
0-0 0 seconds |
7026 |
mo271 author:mo271 |
feat: toMonoidHom_coe |
- [ ] depends on: #6791
---
[](https://gitpod.io/from-referrer/)
|
t-number-theory
merge-conflict
blocked-by-other-PR
|
16/0 |
Mathlib/NumberTheory/LegendreSymbol/MulCharacter.lean |
1 |
3 |
['leanprover-community-mathlib4-bot', 'mo271'] |
nobody |
393-84632 1 year ago |
393-84632 1 year ago |
0-0 0 seconds |
7861 |
shuxuezhuyi author:shuxuezhuyi |
feat(Geometry/Hyperbolic/UpperHalfPlane): instance IsometricSMul PSL(2, ℝ) ℍ |
---
- [ ] depends on: #7835
- [ ] depends on: #7791
[](https://gitpod.io/from-referrer/)
|
t-euclidean-geometry
merge-conflict
blocked-by-other-PR
|
98/0 |
Mathlib.lean,Mathlib/Geometry/Hyperbolic/UpperHalfPlane/Basic.lean,Mathlib/LinearAlgebra/Matrix/ProjectiveSpecialLinearGroup.lean |
3 |
1 |
['leanprover-community-mathlib4-bot'] |
nobody |
369-8268 1 year ago |
369-8268 1 year ago |
0-0 0 seconds |
12087 |
JADekker author:JADekker |
feat : complete API for K-Lindelöf spaces |
---
- [ ] depends on: #11800 (which is now awaiting a design decision)
[](https://gitpod.io/from-referrer/)
|
t-topology
merge-conflict
please-adopt
blocked-by-other-PR
|
789/17 |
Mathlib.lean,Mathlib/Order/Filter/CardinalInter.lean,Mathlib/Topology/Compactness/KLindelof.lean,Mathlib/Topology/Compactness/Lindelof.lean |
4 |
2 |
['github-actions', 'leanprover-community-mathlib4-bot'] |
nobody |
362-20852 11 months ago |
362-20852 11 months ago |
1-72084 1 day |
13782 |
alreadydone author:alreadydone |
feat(EllipticCurve): ZSMul formula in terms of division polynomials |
The formula $[n]P = (\phi_n(x,y) : \omega_n(x,y) : \psi_n(x,y))$ in Jacobian coordinates for $P=(x,y)$ a nonsingular point on a Weierstrass/elliptic curve.
---
- [x] depends on: #12883
- [x] depends on: #13399
- [ ] depends on: #13057
- [ ] depends on: #13155
- [x] depends on: #13845
- [x] depends on: #13846
- [ ] depends on: #13847
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-algebraic-geometry
t-number-theory
merge-conflict
blocked-by-other-PR
label:t-algebra$ |
2462/232 |
Mathlib.lean,Mathlib/Algebra/MvPolynomial/PDeriv.lean,Mathlib/Algebra/Polynomial/Bivariate.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Affine.lean,Mathlib/AlgebraicGeometry/EllipticCurve/DivisionPolynomial/Basic.lean,Mathlib/AlgebraicGeometry/EllipticCurve/DivisionPolynomial/ZSMul.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Group.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Jacobian.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Universal.lean,Mathlib/NumberTheory/EllipticDivisibilitySequence.lean |
10 |
n/a |
['Multramate', 'alreadydone', 'github-actions', 'leanprover-community-mathlib4-bot'] |
nobody |
356-38861 11 months ago |
unknown |
unknown |
14242 |
js2357 author:js2357 |
feat: Prove equivalence of `isDedekindDomain` and `isDedekindDomainDvr` |
Prove that `isDedekindDomainDvr` is equivalent to both `isDedekindDomain` and `isDedekindDomainInv`.
Specifically, prove `isDedekindDomainDvr A → isDedekindDomainInv A`, because `isDedekindDomain A → isDedekindDomainDvr A` and `IsDedekindDomain A ↔ IsDedekindDomainInv A` are already in Mathlib.
- [x] depends on: #14099
- [x] depends on: #14216
- [ ] depends on: #14237
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-algebra
merge-conflict
blocked-by-other-PR
label:t-algebra$ |
269/1 |
Mathlib.lean,Mathlib/RingTheory/DedekindDomain/Dvr.lean,Mathlib/RingTheory/FractionalIdeal/LocalizedAtPrime.lean,Mathlib/RingTheory/Localization/Basic.lean |
4 |
2 |
['github-actions', 'leanprover-community-mathlib4-bot'] |
nobody |
353-58533 11 months ago |
353-58533 11 months ago |
0-0 0 seconds |
16215 |
adomasbaliuka author:adomasbaliuka |
feat(Tactic/Linter): lint unwanted unicode |
Add a text-based style linter that checks all unicode characters.
- Only allow whitelisted characters, with a suggestion to add the flagged character to the whitelist
- Some characters are specified to use emoji-variant or text-variant. The linter ensures these variant-selectors only appear in the correct places and provides an auto-fix to clean them up.
---
Discussed at [Zulip](https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/Whitelist.20for.20Unicode.3F/near/448721083)
The current proposal checks each character against a whitelist. There is also the question of what the whitelist should contain.
A reasonable whitelist might be "all unicode currently in Mathlib" ∪ [Wikipedia/Mathematical_operators_and_symbols_in_Unicode](https://en.wikipedia.org/wiki/Mathematical_operators_and_symbols_in_Unicode) ∪ [EdAyers/mathlib3/docs/unicode.md](https://github.com/EdAyers/mathlib/blob/fb5c2ffe917049959597b0a93b872e91f4004922/docs/unicode.md). Currently implemented is a subset of this list closer to what's currently present in mathlib.
- [x] depends on: #17068
- [x] depends on: #17116
- [ ] depends on: #17129 (part 1 of this PR)
- [ ] depends on: #17131 (part 2 of this PR)
- Future note: @adomasbaliuka says: "we might add something to the Mathlib 4 docs about this as well?"
[](https://gitpod.io/from-referrer/)
|
t-linter
merge-conflict
blocked-by-other-PR
|
462/15 |
Mathlib/GroupTheory/GroupExtension/Defs.lean,Mathlib/Tactic/Linter/TextBased.lean,Mathlib/Tactic/Linter/UnicodeLinter.lean,Mathlib/Tactic/Widget/Calc.lean,Mathlib/Tactic/Widget/CongrM.lean,Mathlib/Tactic/Widget/Conv.lean,Mathlib/Tactic/Widget/GCongr.lean,Mathlib/Topology/ContinuousFunction/Weierstrass.lean,test/LintStyle.lean |
9 |
51 |
['adomasbaliuka', 'eric-wieser', 'github-actions', 'grunweg', 'joneugster', 'mathlib4-dependent-issues-bot'] |
nobody |
348-26542 11 months ago |
348-26542 11 months ago |
12-19694 12 days |
16887 |
metinersin author:metinersin |
feat(ModelTheory/Complexity): define conjunctive and disjunctive formulas |
Defines `FirstOrder.Language.BoundedFormula.IsConjunctive` and `FirstOrder.Language.BoundedFormula.IsDisjunctive`.
---
- [ ] depends on: #16885
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-logic
merge-conflict
blocked-by-other-PR
|
300/7 |
Mathlib/ModelTheory/Complexity.lean,Mathlib/ModelTheory/Equivalence.lean,Mathlib/ModelTheory/Syntax.lean |
3 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
345-54511 11 months ago |
345-54512 11 months ago |
0-1299 21 minutes |
16888 |
metinersin author:metinersin |
feat(ModelTheory/Complexity): Define conjunctive and disjunctive normal forms |
Define `FirstOrder.Language.BoundedFormula.IsDNF` and `FirstOrder.Language.BoundedFormula.IsCNF`.
---
- [ ] depends on: #16887
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-logic
merge-conflict
blocked-by-other-PR
|
415/7 |
Mathlib/ModelTheory/Complexity.lean,Mathlib/ModelTheory/Equivalence.lean,Mathlib/ModelTheory/Syntax.lean |
3 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
345-54511 11 months ago |
345-54511 11 months ago |
0-1045 17 minutes |
16889 |
metinersin author:metinersin |
feat(ModelTheory/Complexity): Normal forms |
Defines `FirstOrder.Language.BoundedFormula.toDNF` and `FirstOrder.Language.BoundedFormula.toCNF` - given a quantifier-free formula, these construct a semantically equivalent formula in disjunctive normal form and conjunctive normal form, respectively.
---
- [ ] depends on: #16888
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-logic
merge-conflict
blocked-by-other-PR
|
525/7 |
Mathlib/ModelTheory/Complexity.lean,Mathlib/ModelTheory/Equivalence.lean,Mathlib/ModelTheory/Syntax.lean |
3 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
345-54510 11 months ago |
345-54510 11 months ago |
0-613 10 minutes |
13965 |
pechersky author:pechersky |
feat(Data/DigitExpansion): reals via digit expansion are complete |
---
[](https://gitpod.io/from-referrer/)
- [ ] depends on: #13964 |
t-data
merge-conflict
blocked-by-other-PR
|
3876/0 |
Mathlib.lean,Mathlib/Data/DigitExpansion/Add.lean,Mathlib/Data/DigitExpansion/Defs.lean,Mathlib/Data/DigitExpansion/Hensel.lean,Mathlib/Data/DigitExpansion/Integer/Basic.lean,Mathlib/Data/DigitExpansion/Integer/Mul.lean,Mathlib/Data/DigitExpansion/Real/Basic.lean,Mathlib/Data/DigitExpansion/Real/CompleteSpace.lean,Mathlib/Data/DigitExpansion/Real/ConditionallyComplete.lean,docs/references.bib |
10 |
4 |
['github-actions', 'leanprover-community-mathlib4-bot'] |
nobody |
332-26252 10 months ago |
332-26252 10 months ago |
0-0 0 seconds |
17519 |
grunweg author:grunweg |
feat: the `metrisableSpace` linter |
Similar to #10235, lint on occurrences of `MetricSpace` which should be `MetrisableSpace`.
---
- [ ] depends on: #10235 (for all the details)
[](https://gitpod.io/from-referrer/)
|
t-linter
merge-conflict
blocked-by-other-PR
|
155/21 |
Mathlib.lean,Mathlib/Algebra/MvPolynomial/PDeriv.lean,Mathlib/AlgebraicGeometry/EllipticCurve/NormalForms.lean,Mathlib/Computability/Halting.lean,Mathlib/Computability/TuringMachine.lean,Mathlib/Data/Fintype/Card.lean,Mathlib/Data/MLList/Split.lean,Mathlib/GroupTheory/Perm/DomMulAct.lean,Mathlib/Logic/Basic.lean,Mathlib/Logic/Encodable/Basic.lean,Mathlib/MeasureTheory/Covering/VitaliFamily.lean,Mathlib/MeasureTheory/Measure/Doubling.lean,Mathlib/NumberTheory/JacobiSum/Basic.lean,Mathlib/Order/Heyting/Regular.lean,Mathlib/Tactic.lean,Mathlib/Tactic/FunProp/RefinedDiscrTree.lean,Mathlib/Tactic/Linter/UnusedAssumptionInType.lean,Mathlib/Util/Superscript.lean,scripts/noshake.json |
19 |
4 |
['github-actions', 'mathlib4-dependent-issues-bot', 'urkud'] |
nobody |
331-49166 10 months ago |
340-49640 11 months ago* |
340-49610 340 days* |
12750 |
Command-Master author:Command-Master |
feat: define Gray code |
---
Define binary reflected gray code, both as a permutation of `Nat` and as a permutation of `BitVec n`, and prove some theorems about them. Additionally, remove `@[simp]` from `Nat.bit_false` and `Nat.bit_true`, as `bit0` and `bit1` are deprecated, and add some lemmas to `Bits`, `Bitwise` and `Size`.
- [ ] depends on: #12751
[](https://gitpod.io/from-referrer/)
|
t-data
new-contributor
merge-conflict
awaiting-author
blocked-by-other-PR
|
226/0 |
Mathlib.lean,Mathlib/Data/Nat/Bits.lean,Mathlib/Data/Nat/Bitwise.lean,Mathlib/Data/Nat/GrayCode.lean,Mathlib/Data/Nat/Size.lean |
5 |
5 |
['Rida-Hamadani', 'alreadydone', 'github-actions', 'grunweg', 'leanprover-community-mathlib4-bot'] |
nobody |
327-77168 10 months ago |
327-77168 10 months ago |
6-8380 6 days |
13514 |
madvorak author:madvorak |
feat(Computability/ContextFreeGrammar): closure under union |
- [ ] depends on: #15895
---
[](https://gitpod.io/from-referrer/)
|
t-computability
merge-conflict
blocked-by-other-PR
|
448/4 |
Mathlib/Computability/ContextFreeGrammar.lean |
1 |
50 |
['Rida-Hamadani', 'YaelDillies', 'github-actions', 'leanprover-community-mathlib4-bot', 'madvorak'] |
nobody |
315-2096 10 months ago |
315-2096 10 months ago |
72-28392 72 days |
17518 |
grunweg author:grunweg |
feat: lint on declarations mentioning `Invertible` or `Unique` |
Using the same infrastructure as for #10235. Depends on that PR to land first, and also (for the first lint) a zulip discussion if that change is desired/about the best way to enact it.
---
- [ ] depends on: #10235 |
awaiting-zulip
t-linter
merge-conflict
blocked-by-other-PR
|
149/7 |
Mathlib.lean,Mathlib/Algebra/MvPolynomial/PDeriv.lean,Mathlib/Computability/Halting.lean,Mathlib/Computability/TuringMachine.lean,Mathlib/Data/Fintype/Card.lean,Mathlib/GroupTheory/Perm/DomMulAct.lean,Mathlib/Logic/Basic.lean,Mathlib/Logic/Encodable/Basic.lean,Mathlib/NumberTheory/JacobiSum/Basic.lean,Mathlib/Order/Heyting/Regular.lean,Mathlib/RingTheory/MvPolynomial/Symmetric/FundamentalTheorem.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter/UnusedAssumptionInType.lean |
13 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mergify'] |
nobody |
314-61229 10 months ago |
340-49751 11 months ago* |
0-0 0 seconds* |
16428 |
FR-vdash-bot author:FR-vdash-bot |
test use `QuotLike` APIs |
---
- [ ] depends on: #16421
[](https://gitpod.io/from-referrer/)
|
t-data
merge-conflict
blocked-by-other-PR
|
1501/564 |
Mathlib.lean,Mathlib/Algebra/Associated/Basic.lean,Mathlib/Algebra/BigOperators/Associated.lean,Mathlib/Algebra/GCDMonoid/Basic.lean,Mathlib/Algebra/Group/Conj.lean,Mathlib/Algebra/GroupWithZero/NonZeroDivisors.lean,Mathlib/Algebra/Order/CauSeq/Completion.lean,Mathlib/Algebra/Quandle.lean,Mathlib/CategoryTheory/IsomorphismClasses.lean,Mathlib/CategoryTheory/Monoidal/Free/Basic.lean,Mathlib/CategoryTheory/Monoidal/Free/Coherence.lean,Mathlib/CategoryTheory/Skeletal.lean,Mathlib/Data/Finmap.lean,Mathlib/Data/Fintype/Quotient.lean,Mathlib/Data/Multiset/Basic.lean,Mathlib/Data/Multiset/Functor.lean,Mathlib/Data/QPF/Multivariate/Constructions/Fix.lean,Mathlib/Data/QPF/Univariate/Basic.lean,Mathlib/Data/Quot.lean,Mathlib/Data/QuotLike.lean,Mathlib/Data/Real/Basic.lean,Mathlib/Data/Setoid/Basic.lean,Mathlib/GroupTheory/Coset/Basic.lean,Mathlib/GroupTheory/Coset/Defs.lean,Mathlib/GroupTheory/GroupAction/Basic.lean,Mathlib/GroupTheory/GroupAction/ConjAct.lean,Mathlib/GroupTheory/GroupAction/Defs.lean,Mathlib/GroupTheory/QuotientGroup/Basic.lean,Mathlib/GroupTheory/QuotientGroup/Defs.lean,Mathlib/GroupTheory/Subgroup/Center.lean,Mathlib/LinearAlgebra/Quotient/Basic.lean,Mathlib/LinearAlgebra/Quotient/Defs.lean,Mathlib/Logic/Encodable/Basic.lean,Mathlib/Logic/Equiv/Basic.lean,Mathlib/Logic/Relation.lean,Mathlib/Order/RelIso/Basic.lean,Mathlib/SetTheory/Cardinal/Basic.lean,Mathlib/SetTheory/Cardinal/Finite.lean,Mathlib/SetTheory/Game/Basic.lean,Mathlib/SetTheory/Lists.lean,Mathlib/SetTheory/ZFC/Basic.lean,Mathlib/Topology/Inseparable.lean,test/QuotLike.lean |
43 |
2 |
['github-actions', 'leanprover-community-mathlib4-bot'] |
nobody |
312-76308 10 months ago |
312-76308 10 months ago |
0-0 0 seconds |
18716 |
jjaassoonn author:jjaassoonn |
feat(Algebra/Module/GradedModule): quotient and subgrading |
- [ ] depends on: #9820
[](https://gitpod.io/from-referrer/)
|
t-algebra
awaiting-CI
merge-conflict
blocked-by-other-PR
WIP
label:t-algebra$ |
997/191 |
Counterexamples/HomogeneousPrimeNotPrime.lean,Mathlib.lean,Mathlib/Algebra/Group/Subgroup/Defs.lean,Mathlib/Algebra/Module/GradedModule/Basic.lean,Mathlib/Algebra/Module/GradedModule/QuotientGrading.lean,Mathlib/Algebra/Module/GradedModule/Subgrading.lean,Mathlib/AlgebraicGeometry/ProjectiveSpectrum/Topology.lean,Mathlib/RingTheory/GradedAlgebra/Homogeneous/Ideal.lean,Mathlib/RingTheory/GradedAlgebra/Homogeneous/Submodule.lean,Mathlib/RingTheory/GradedAlgebra/Quotient.lean,Mathlib/RingTheory/GradedAlgebra/Radical.lean,scripts/no_lints_prime_decls.txt |
12 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
308-61196 10 months ago |
308-61196 10 months ago |
0-0 0 seconds |
18784 |
erdOne author:erdOne |
feat(AlgebraicGeometry) use `addMorphismPropertyInstances` |
---
- [ ] depends on: #18785
[](https://gitpod.io/from-referrer/)
|
t-algebraic-geometry
merge-conflict
blocked-by-other-PR
|
435/91 |
Mathlib.lean,Mathlib/AlgebraicGeometry/Cover/Open.lean,Mathlib/AlgebraicGeometry/Morphisms/Affine.lean,Mathlib/AlgebraicGeometry/Morphisms/ClosedImmersion.lean,Mathlib/AlgebraicGeometry/Morphisms/FinitePresentation.lean,Mathlib/AlgebraicGeometry/Morphisms/FiniteType.lean,Mathlib/AlgebraicGeometry/Morphisms/OpenImmersion.lean,Mathlib/AlgebraicGeometry/Morphisms/Proper.lean,Mathlib/AlgebraicGeometry/Morphisms/QuasiCompact.lean,Mathlib/AlgebraicGeometry/Morphisms/QuasiSeparated.lean,Mathlib/AlgebraicGeometry/Morphisms/RingHomProperties.lean,Mathlib/AlgebraicGeometry/Morphisms/Smooth.lean,Mathlib/AlgebraicGeometry/Morphisms/UniversallyClosed.lean,Mathlib/AlgebraicGeometry/Restrict.lean,Mathlib/CategoryTheory/MorphismProperty/Composition.lean,Mathlib/CategoryTheory/MorphismProperty/Limits.lean,Mathlib/CategoryTheory/MorphismProperty/Tactic.lean,MathlibTest/AddMorphismPropertyInstances.lean |
18 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
308-217 10 months ago |
308-217 10 months ago |
0-1869 31 minutes |
16014 |
vihdzp author:vihdzp |
feat(SetTheory/Ordinal/Principal): even more lemmas on additively principal ordinals |
---
These are useful for my work on Cantor normal forms.
- [ ] depends on: #15989
[](https://gitpod.io/from-referrer/)
|
t-set-theory
t-logic
merge-conflict
blocked-by-other-PR
|
99/60 |
Mathlib/SetTheory/Ordinal/Exponential.lean,Mathlib/SetTheory/Ordinal/Principal.lean |
2 |
2 |
['github-actions', 'leanprover-community-mathlib4-bot'] |
nobody |
304-84659 10 months ago |
304-84659 10 months ago |
0-664 11 minutes |
17593 |
FR-vdash-bot author:FR-vdash-bot |
chore(Algebra/Order/GroupWithZero/Unbundled): deprecate useless lemmas, use `ZeroLEOneClass` |
There are still some useless lemmas that were simply ported from `Algebra.Order.Monoid.Lemmas`, such as just chain an existing lemma with an assumption and lemmas whose assumptions imply `1 ≤ 0`. This PR removes them.
Also, some lemmas have both assumptions like `1 < a` `0 < a`. This PR uses `ZeroLEOneClass` to remove redundant assumptions.
---
- [ ] depends on: #17623
Ported from https://github.com/leanprover-community/mathlib/pull/16525 and https://github.com/leanprover-community/mathlib/pull/18158
Adapted from #9250. This version is easier to review.
[](https://gitpod.io/from-referrer/)
|
t-order
t-algebra
merge-conflict
blocked-by-other-PR
label:t-algebra$ |
188/48 |
Archive/Wiedijk100Theorems/BuffonsNeedle.lean,Mathlib/Algebra/Order/GroupWithZero/Canonical.lean,Mathlib/Algebra/Order/GroupWithZero/Unbundled.lean,Mathlib/Combinatorics/SimpleGraph/Triangle/Counting.lean,Mathlib/RingTheory/DedekindDomain/FiniteAdeleRing.lean,Mathlib/Topology/Algebra/Order/Field.lean |
6 |
n/a |
['FR-vdash-bot', 'github-actions', 'mathlib4-dependent-issues-bot', 'vihdzp'] |
nobody |
296-80760 9 months ago |
unknown |
unknown |
17624 |
FR-vdash-bot author:FR-vdash-bot |
feat(Algebra/Order/GroupWithZero/Unbundled): generalize lemmas |
---
- [ ] depends on: #17623
[](https://gitpod.io/from-referrer/)
|
t-order
t-algebra
merge-conflict
blocked-by-other-PR
label:t-algebra$ |
121/26 |
Mathlib/Algebra/Order/GroupWithZero/Unbundled.lean |
1 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
293-31532 9 months ago |
293-31532 9 months ago |
0-465 7 minutes |
17515 |
FR-vdash-bot author:FR-vdash-bot |
perf: do not need `simp low` now |
---
- [ ] depends on: #17513
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
blocked-by-other-PR
label:t-algebra$ |
12/10 |
Mathlib/Algebra/Group/Hom/Defs.lean,Mathlib/Analysis/SpecialFunctions/Bernstein.lean,Mathlib/GroupTheory/GroupAction/Hom.lean,Mathlib/NumberTheory/LucasLehmer.lean |
4 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
291-76953 9 months ago |
291-76953 9 months ago |
0-380 6 minutes |
16210 |
FR-vdash-bot author:FR-vdash-bot |
Clean up quotient APIs |
~~We may migrate to `Quot` and `IsEquiv` APIs in the future, but it might be a good start to clean up `Quotient` APIs anyway.~~
The diffs in this PR did not include `QuotLike` APIs, but eventually I decided to migrate to `QuotLike` before deprecating some old APIs. This is because some lemmas don't have alternatives that don't use `· ≈ ·`, and the alternatives that use `· ≈ ·` are in the core. See [Zulip](https://leanprover.zulipchat.com/#narrow/stream/113488-general/topic/.60.28.C2.B7.20.E2.89.88.20.C2.B7.29.60.20in.20.60Quotient.60.20APIs/near/466970386).
---
- [x] depends on: #16254
- [x] depends on: #16256
- [x] depends on: #16258
- [x] depends on: #16260
- [x] depends on: #16264
- [x] depends on: #16267
- [ ] depends on: #16314
- [x] depends on: #16410
- [x] depends on: #17588
- [x] depends on: #17594
- [x] depends on: #17940
- [ ] depends on: #17941
---
`QuotLike`
- [ ] depends on: #16421
- [ ] depends on: #16428
---
[remaining diffs](https://github.com/leanprover-community/mathlib4/compare/FR_quot_now..FR_quot)
[](https://gitpod.io/from-referrer/)
|
t-data
tech debt
merge-conflict
blocked-by-other-PR
|
1015/1114 |
Counterexamples/CliffordAlgebraNotInjective.lean,Mathlib/Algebra/Associated/Basic.lean,Mathlib/Algebra/BigOperators/Group/Finset.lean,Mathlib/Algebra/CharZero/Quotient.lean,Mathlib/Algebra/DirectLimit.lean,Mathlib/Algebra/GCDMonoid/Basic.lean,Mathlib/Algebra/Lie/Free.lean,Mathlib/Algebra/Lie/Quotient.lean,Mathlib/Algebra/Module/Torsion.lean,Mathlib/Algebra/Module/Zlattice/Basic.lean,Mathlib/Algebra/Order/CauSeq/Completion.lean,Mathlib/Algebra/Periodic.lean,Mathlib/Algebra/RingQuot.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Jacobian.lean,Mathlib/AlgebraicGeometry/ProjectiveSpectrum/Scheme.lean,Mathlib/AlgebraicGeometry/ProjectiveSpectrum/StructureSheaf.lean,Mathlib/Analysis/Normed/Group/Quotient.lean,Mathlib/Analysis/Normed/Group/SemiNormedGrp/Kernels.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Angle.lean,Mathlib/CategoryTheory/ConnectedComponents.lean,Mathlib/CategoryTheory/Limits/Shapes/SingleObj.lean,Mathlib/CategoryTheory/Limits/Types.lean,Mathlib/CategoryTheory/Skeletal.lean,Mathlib/CategoryTheory/Subobject/Basic.lean,Mathlib/CategoryTheory/Subobject/FactorThru.lean,Mathlib/CategoryTheory/Subobject/Lattice.lean,Mathlib/Combinatorics/Quiver/ConnectedComponent.lean,Mathlib/Combinatorics/SimpleGraph/Path.lean,Mathlib/Computability/Reduce.lean,Mathlib/Computability/TuringMachine.lean,Mathlib/Data/Countable/Defs.lean,Mathlib/Data/FinEnum.lean,Mathlib/Data/Finite/Basic.lean,Mathlib/Data/Fintype/Basic.lean,Mathlib/Data/Fintype/Card.lean,Mathlib/Data/Fintype/Quotient.lean,Mathlib/Data/List/Cycle.lean,Mathlib/Data/Multiset/Basic.lean,Mathlib/Data/Quot.lean,Mathlib/Data/Set/Image.lean,Mathlib/Data/Setoid/Basic.lean,Mathlib/Data/Setoid/Partition.lean,Mathlib/Data/Sym/Sym2.lean,Mathlib/FieldTheory/IsAlgClosed/AlgebraicClosure.lean,Mathlib/FieldTheory/PerfectClosure.lean,Mathlib/FieldTheory/SplittingField/Construction.lean,Mathlib/GroupTheory/Abelianization.lean,Mathlib/GroupTheory/Commensurable.lean,Mathlib/GroupTheory/CommutingProbability.lean,Mathlib/GroupTheory/Complement.lean,Mathlib/GroupTheory/Congruence/Basic.lean,Mathlib/GroupTheory/Coprod/Basic.lean,Mathlib/GroupTheory/Coset/Basic.lean,Mathlib/GroupTheory/DoubleCoset.lean,Mathlib/GroupTheory/FreeAbelianGroup.lean,Mathlib/GroupTheory/GroupAction/Basic.lean,Mathlib/GroupTheory/GroupAction/ConjAct.lean,Mathlib/GroupTheory/GroupAction/Quotient.lean,Mathlib/GroupTheory/Index.lean,Mathlib/GroupTheory/MonoidLocalization/Basic.lean,Mathlib/GroupTheory/Nilpotent.lean,Mathlib/GroupTheory/PGroup.lean,Mathlib/GroupTheory/Perm/Cycle/Concrete.lean,Mathlib/GroupTheory/QuotientGroup/Basic.lean,Mathlib/GroupTheory/SchurZassenhaus.lean,Mathlib/GroupTheory/Sylow.lean,Mathlib/GroupTheory/Transfer.lean,Mathlib/LinearAlgebra/Alternating/DomCoprod.lean,Mathlib/LinearAlgebra/Dimension/Constructions.lean,Mathlib/LinearAlgebra/InvariantBasisNumber.lean,Mathlib/LinearAlgebra/Isomorphisms.lean,Mathlib/LinearAlgebra/Projectivization/Basic.lean,Mathlib/LinearAlgebra/Quotient.lean,Mathlib/LinearAlgebra/QuotientPi.lean,Mathlib/Logic/Encodable/Basic.lean,Mathlib/MeasureTheory/Constructions/Polish/Basic.lean,Mathlib/MeasureTheory/Function/AEEqFun.lean,Mathlib/MeasureTheory/Group/FundamentalDomain.lean,Mathlib/MeasureTheory/MeasurableSpace/Basic.lean,Mathlib/MeasureTheory/Measure/Haar/Quotient.lean,Mathlib/ModelTheory/DirectLimit.lean,Mathlib/ModelTheory/Fraisse.lean,Mathlib/ModelTheory/Ultraproducts.lean,Mathlib/NumberTheory/NumberField/Embeddings.lean,Mathlib/NumberTheory/NumberField/Units/DirichletTheorem.lean,Mathlib/NumberTheory/Padics/PadicNumbers.lean,Mathlib/NumberTheory/RamificationInertia.lean,Mathlib/Order/Antisymmetrization.lean,Mathlib/Order/Category/PartOrd.lean,Mathlib/Order/Filter/Germ/Basic.lean,Mathlib/Order/Partition/Finpartition.lean,Mathlib/Order/RelIso/Basic.lean,Mathlib/RepresentationTheory/GroupCohomology/Hilbert90.lean,Mathlib/RingTheory/AdicCompletion/Algebra.lean,Mathlib/RingTheory/AdicCompletion/Basic.lean,Mathlib/RingTheory/AdicCompletion/Functoriality.lean,Mathlib/RingTheory/AdjoinRoot.lean,Mathlib/RingTheory/Congruence/Basic.lean,Mathlib/RingTheory/Flat/Basic.lean,Mathlib/RingTheory/GradedAlgebra/HomogeneousLocalization.lean |
134 |
6 |
['FR-vdash-bot', 'github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot'] |
nobody |
287-65417 9 months ago |
375-54498 1 year ago |
0-0 0 seconds |
19414 |
vihdzp author:vihdzp |
feat: Nesbitt's inequality |
We prove [Nesbitt's inequality](https://en.wikipedia.org/wiki/Nesbitt%27s_inequality) `3 / 2 ≤ a / (b + c) + b / (c + a) + c / (b + a)` for a linearly ordered semifield, by reduction to the AM-HM inequality.
---
- [ ] depends on: #19415
- [ ] depends on: #19420
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebra
merge-conflict
awaiting-author
blocked-by-other-PR
WIP
label:t-algebra$ |
192/142 |
Mathlib/Algebra/BigOperators/Fin.lean,Mathlib/Algebra/BigOperators/Finsupp.lean,Mathlib/Algebra/Order/Antidiag/Pi.lean,Mathlib/Algebra/Order/BigOperators/Ring/Finset.lean,Mathlib/Algebra/Order/Field/Defs.lean,Mathlib/Analysis/MeanInequalities.lean,Mathlib/Combinatorics/Enumerative/Catalan.lean,Mathlib/Data/Fin/Tuple/NatAntidiagonal.lean,Mathlib/Data/Fin/Tuple/Reflection.lean,Mathlib/Data/Fintype/BigOperators.lean |
10 |
8 |
['YaelDillies', 'github-actions', 'mathlib4-dependent-issues-bot', 'vihdzp'] |
nobody |
285-27277 9 months ago |
285-27277 9 months ago |
0-481 8 minutes |
18876 |
GabinKolly author:GabinKolly |
feat(ModelTheory/Fraisse): add proof that Fraïssé limits exist |
Fraïssé limits exist.
---
All the preparatory work done in other files is contained in the pull request #18749, this pull request adds the work done in ModelTheory/Fraisse, the definition of the sequence of structures whose limit will be the Fraïssé limit, lemmas about this sequence, and then the proof that the limit is indeed a Fraïssé limit.
- [ ] depends on: #18749
[](https://gitpod.io/from-referrer/)
|
t-logic
blocked-by-other-PR
|
666/5 |
Mathlib/ModelTheory/Bundled.lean,Mathlib/ModelTheory/DirectLimit.lean,Mathlib/ModelTheory/FinitelyGenerated.lean,Mathlib/ModelTheory/Fraisse.lean,Mathlib/ModelTheory/PartialEquiv.lean,Mathlib/ModelTheory/Substructures.lean |
6 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
279-78992 9 months ago |
305-68962 10 months ago |
0-37 37 seconds |
19281 |
Vierkantor author:Vierkantor |
chore(Algebra/{MonoidAlgebra,Polynomial}): algebra structure in `Basic.lean` |
[As discussed in PR 19205](https://github.com/leanprover-community/mathlib4/pull/19205#discussion_r1848539148) the Algebra structure on `Polynomial` and `MonoidAlgebra` is very fundamental and shouldn't be hidden away. So let's refactor the import hierarchy to make them available in `Basic.lean`.
In addition to #19097, this moves the algebra structure on polynomials into `Algebra/Polynomial/Basic.lean` (which will import the other important instances on polynomials), and moves the algebra structure on `MonoidAlgebra`s into `Algebra/MonoidAlgebra/Basic.lean` (moving most of the existing results in that file into `Lemmas.lean`).
---
- [ ] depends on: #19097
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
blocked-by-other-PR
label:t-algebra$ |
3506/2792 |
Counterexamples/ZeroDivisorsInAddMonoidAlgebras.lean,Mathlib.lean,Mathlib/Algebra/BigOperators/Finsupp.lean,Mathlib/Algebra/FreeAlgebra.lean,Mathlib/Algebra/FreeNonUnitalNonAssocAlgebra.lean,Mathlib/Algebra/MonoidAlgebra/Basic.lean,Mathlib/Algebra/MonoidAlgebra/Defs.lean,Mathlib/Algebra/MonoidAlgebra/Division.lean,Mathlib/Algebra/MonoidAlgebra/Lemmas.lean,Mathlib/Algebra/MonoidAlgebra/Lift.lean,Mathlib/Algebra/MonoidAlgebra/MapDomain.lean,Mathlib/Algebra/MonoidAlgebra/Module.lean,Mathlib/Algebra/MonoidAlgebra/Opposite.lean,Mathlib/Algebra/MonoidAlgebra/Support.lean,Mathlib/Algebra/MvPolynomial/Basic.lean,Mathlib/Algebra/Polynomial/AlgebraMap.lean,Mathlib/Algebra/Polynomial/Basic.lean,Mathlib/Algebra/Polynomial/Cardinal.lean,Mathlib/Algebra/Polynomial/Coeff.lean,Mathlib/Algebra/Polynomial/Defs.lean,Mathlib/Algebra/Polynomial/Degree/Definitions.lean,Mathlib/Algebra/Polynomial/Degree/TrailingDegree.lean,Mathlib/Algebra/Polynomial/EraseUpdate.lean,Mathlib/Algebra/Polynomial/Eval/Defs.lean,Mathlib/Algebra/Polynomial/Eval/Degree.lean,Mathlib/Algebra/Polynomial/Laurent.lean,Mathlib/Algebra/Polynomial/Module.lean,Mathlib/Algebra/Polynomial/Monomial.lean,Mathlib/Algebra/Polynomial/Sum.lean,Mathlib/Algebra/Polynomial/Taylor.lean,Mathlib/Data/Finsupp/Basic.lean,Mathlib/Data/Finsupp/Defs.lean,Mathlib/Data/Finsupp/Ext.lean,Mathlib/Data/Finsupp/Fintype.lean,Mathlib/Data/Finsupp/Indicator.lean,Mathlib/Data/Finsupp/Notation.lean,Mathlib/Data/Finsupp/Pointwise.lean,Mathlib/Data/Finsupp/SMulWithZero.lean,Mathlib/Data/Finsupp/Single.lean,Mathlib/Data/List/ToFinsupp.lean,Mathlib/LinearAlgebra/Matrix/Charpoly/Eigs.lean,Mathlib/RepresentationTheory/Maschke.lean,Mathlib/RingTheory/FiniteType.lean,Mathlib/RingTheory/KrullDimension/Basic.lean,Mathlib/RingTheory/MvPolynomial/Basic.lean,Mathlib/RingTheory/Polynomial/Opposites.lean,Mathlib/RingTheory/Polynomial/Wronskian.lean,Mathlib/RingTheory/PowerSeries/Basic.lean,Mathlib/Tactic/ExtractGoal.lean,MathlibTest/Polynomial.lean,MathlibTest/instance_diamonds.lean,scripts/noshake.json |
52 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
276-79122 9 months ago |
286-56252 9 months ago |
0-0 0 seconds |
19621 |
Command-Master author:Command-Master |
feat: Multiplicity and prime-adic valuation of derivations |
---
- [ ] depends on: #19596
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebra
merge-conflict
blocked-by-other-PR
label:t-algebra$ |
397/13 |
Mathlib.lean,Mathlib/Algebra/Order/AddGroupWithTop.lean,Mathlib/Algebra/Order/Monoid/Unbundled/WithTop.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/Order/WithBot.lean,Mathlib/RingTheory/Derivation/Multiplicity.lean,Mathlib/RingTheory/DiscreteValuationRing/Basic.lean,Mathlib/RingTheory/Valuation/Basic.lean,Mathlib/RingTheory/Valuation/PrimeMultiplicity.lean |
9 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
266-75820 8 months ago |
266-75820 8 months ago |
0-666 11 minutes |
18262 |
joelriou author:joelriou |
feat(Algebra/Category/ModuleCat/Presheaf): exterior powers of presheaves of modules |
---
- [x] depends on: #18261
- [ ] depends on: #18236
- [ ] depends on: #18197
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-category-theory
merge-conflict
blocked-by-other-PR
WIP
label:t-algebra$ |
874/0 |
Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/ChangeOfRings.lean,Mathlib/Algebra/Category/ModuleCat/ExteriorPower.lean,Mathlib/Algebra/Category/ModuleCat/Presheaf/ExteriorPower.lean,Mathlib/Algebra/Category/ModuleCat/Presheaf/FunctorOfNatTrans.lean,Mathlib/Algebra/Category/ModuleCat/Pseudofunctor.lean |
6 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
266-67115 8 months ago |
302-47180 9 months ago |
0-0 0 seconds |
11156 |
smorel394 author:smorel394 |
feat(LinearAlgebra/{TensorProductBasis,Dual}): basis and dual of `PiTensorProduct` |
Construct a basis of a `PiTensorProduct` of modules given bases of the modules, and relationship between the dual of a `PiTensorProduct` and the `PiTensorProduct` of the duals.
Main results:
* `Basis.piTensorProduct` (in `LinearAlgebra/TensorProductBasis.lean`): Let `ι` be a `Fintype` and `M` be a family of modules indexed by `ι`. If `b i : κ i → M i` is a basis for every `i` in `ι`, then `fun (p : Π i, κ i) ↦ ⨂ₜ[R] i, b i (p i)` is a basis of `⨂[R] i, M i`.
* `PiTensorProduct.dualDistrib` (in `LinearAlgebra/Dual.lean`): The canonical linear map from `⨂[R] i, Dual R (M i)` to `Dual R (⨂[R] i, M i)`, sending `⨂ₜ[R] i, f i` to the composition of `PiTensorProduct.map f` with the linear equivalence `⨂[R] i, R →ₗ R` given by multiplication.
* `PiTensorProduct.dualDistribEquiv` (also in `LinearAlgebra/Dual.lean`): A linear equivalence between `⨂[R] i, Dual R (M i)` and `Dual R (⨂[R] i, M i)` when all `M i` are finite free modules. If `f : (i : ι) → Dual R (M i)`, then this equivalence sends `⨂ₜ[R] i, f i` to the composition of `PiTensorProduct.map f` with the natural isomorphism `⨂[R] i, R ≃ R` given by multiplication.
- [ ] depends on: #11155 (currently used as the base branch; do not merge without switching it back to `master`!)
---
[](https://gitpod.io/from-referrer/)
|
large-import
new-contributor
t-algebra
merge-conflict
please-adopt
blocked-by-other-PR
label:t-algebra$ |
166/2 |
Mathlib/LinearAlgebra/DirectSum/Finsupp.lean,Mathlib/LinearAlgebra/Dual.lean,Mathlib/LinearAlgebra/TensorProduct/Basis.lean |
3 |
4 |
['eric-wieser', 'github-actions', 'leanprover-community-mathlib4-bot'] |
nobody |
256-75245 8 months ago |
302-4473 9 months ago |
0-0 0 seconds |
15269 |
kkytola author:kkytola |
feat: Add ENNReal.floor |
A right-continuous floor function on `ENNReal`.
---
- [x] depends on: #13938
- [ ] depends on: #15773 (general type class for `ENat`-valued floor functions)
- [x] depends on: #15380 (topology on `ENat` is needed to state right continuity of the floor function)
[](https://gitpod.io/from-referrer/)
|
t-order
t-algebra
merge-conflict
awaiting-author
blocked-by-other-PR
label:t-algebra$ |
445/0 |
Mathlib.lean,Mathlib/Algebra/Order/EFloor.lean,Mathlib/Data/ENNReal/Floor.lean,Mathlib/Data/Nat/Lattice.lean |
4 |
18 |
['YaelDillies', 'github-actions', 'kkytola', 'leanprover-community-mathlib4-bot', 'urkud'] |
nobody |
253-48049 8 months ago |
253-48049 8 months ago |
0-3440 57 minutes |
17471 |
joelriou author:joelriou |
feat(Algebra/ModuleCat/Differentials/Sheaf): the sheaf of relative differentials |
---
- [ ] depends on: #17366
- [x] depends on: #17388
- [x] depends on: #16755
- [ ] depends on: #17469
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebraic-geometry
t-category-theory
merge-conflict
blocked-by-other-PR
WIP
|
740/10 |
Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Differentials/Presheaf.lean,Mathlib/Algebra/Category/ModuleCat/Differentials/Sheaf.lean,Mathlib/Algebra/Category/ModuleCat/Presheaf/Limits.lean,Mathlib/Algebra/Category/ModuleCat/Presheaf/Pullback.lean,Mathlib/Algebra/Category/Ring/Constructions.lean,Mathlib/Algebra/Ring/Hom/Defs.lean,Mathlib/AlgebraicGeometry/Modules/Differentials.lean,Mathlib/Geometry/RingedSpace/SheafedSpace.lean |
9 |
n/a |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
244-62466 8 months ago |
unknown |
unknown |
19462 |
joelriou author:joelriou |
feat(AlgebraicGeometry): étale sheafification |
After #19096 and #18945 are merged, if `S : Scheme.{u}`, we shall get instances like `HasSheafify (smallEtaleTopology S) (Type (u + 1))` which means that in order to sheafify preshaves over the small étale site of `S`, we need to assume a certain bump in the universe in the target category.
With the main result in this PR (there are still a few sorries), we shall get `HasSheafify (smallEtaleTopology S) (Type u)`. Then, in the subsequent development of étale formalism, we can work in `Type u` (or `Ab.{u}`, etc).
---
This is a draft.
- [ ] depends on: #19444
[](https://gitpod.io/from-referrer/)
|
t-algebraic-geometry
merge-conflict
blocked-by-other-PR
WIP
|
1336/2 |
Mathlib.lean,Mathlib/AlgebraicGeometry/Sites/EtaleSheafification.lean,Mathlib/CategoryTheory/Sites/Continuous.lean,Mathlib/CategoryTheory/Sites/DenseSubsite.lean,Mathlib/CategoryTheory/Sites/LocallyFullyFaithful.lean,Mathlib/CategoryTheory/Sites/OneHypercover.lean,Mathlib/CategoryTheory/Sites/OneHypercoverDense.lean,Mathlib/CategoryTheory/Sites/Sieves.lean |
8 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
242-74924 7 months ago |
289-83061 9 months ago |
0-200 3 minutes |
15720 |
znssong author:znssong |
feat(SimpleGraph): The Bondy-Chvátal theorem |
The proof of the Bondy-Chvátal theorem, with Dirac's theorem and Ore's theorem as its corollary.
- [x] depends on: #15536
- [ ] depends on: #15711
- [ ] depends on: #15578 |
new-contributor
t-combinatorics
merge-conflict
blocked-by-other-PR
|
903/3 |
Mathlib.lean,Mathlib/Combinatorics/SimpleGraph/BondyChvatal.lean,Mathlib/Combinatorics/SimpleGraph/Finite.lean,Mathlib/Combinatorics/SimpleGraph/Hamiltonian.lean,Mathlib/Combinatorics/SimpleGraph/Path.lean,Mathlib/Combinatorics/SimpleGraph/Walk.lean,Mathlib/Dynamics/FixedPoints/Basic.lean,Mathlib/Dynamics/FixedPoints/Increasing.lean |
8 |
3 |
['github-actions', 'grunweg', 'leanprover-community-mathlib4-bot'] |
YaelDillies assignee:YaelDillies |
239-77512 7 months ago |
239-77512 7 months ago |
0-1791 29 minutes |
14412 |
jjaassoonn author:jjaassoonn |
feat: show stalk of presheaf of modules is a module over stalk of ring |
---
- [x] depends on: #14413
- [ ] depends on: #14501
[](https://gitpod.io/from-referrer/)
|
workshop-AIM-AG-2024
t-algebraic-geometry
merge-conflict
blocked-by-other-PR
|
966/2 |
Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Presheaf/OverColimitsRing'.lean,Mathlib/Algebra/Category/ModuleCat/Presheaf/OverColimitsRing.lean,Mathlib/CategoryTheory/Filtered/Basic.lean,Mathlib/CategoryTheory/Limits/ConcreteCategory.lean,Mathlib/Geometry/RingedSpace/Basic.lean,Mathlib/Geometry/RingedSpace/Module.lean,Mathlib/Topology/Sheaves/Stalks.lean |
8 |
5 |
['github-actions', 'jjaassoonn', 'leanprover-community-mathlib4-bot', 'smorel394'] |
nobody |
237-62014 7 months ago |
393-85634 1 year ago |
0-0 0 seconds |
12670 |
trivial1711 author:trivial1711 |
feat: completion of a nonarchimedean multiplicative group |
We prove that the completion of a nonarchimedean multiplicative group is a nonarchimedean multiplicative group.
---
- [x] depends on: #12669
- [ ] depends on: #11837
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-topology
merge-conflict
blocked-by-other-PR
label:t-algebra$ |
358/228 |
Mathlib/Analysis/InnerProductSpace/Completion.lean,Mathlib/Analysis/Normed/Group/HomCompletion.lean,Mathlib/Analysis/Normed/Module/Completion.lean,Mathlib/Topology/Algebra/GroupCompletion.lean,Mathlib/Topology/Algebra/InfiniteSum/GroupCompletion.lean,Mathlib/Topology/Algebra/Nonarchimedean/Completion.lean,Mathlib/Topology/Algebra/UniformField.lean,Mathlib/Topology/Algebra/UniformMulAction.lean,Mathlib/Topology/Algebra/UniformRing.lean |
9 |
n/a |
['github-actions', 'leanprover-community-mathlib4-bot'] |
nobody |
225-50413 7 months ago |
unknown |
unknown |
21277 |
GabinKolly author:GabinKolly |
feat(ModelTheory/PartialEquiv): Define the mapping of a self-partialEquiv through an embedding |
Define the mapping of a self-partialEquiv through an embedding and the notion of fully extendable partialEquiv.
---
This is some preparatory work for #18876
- [ ] depends on: #21276
[](https://gitpod.io/from-referrer/)
|
t-logic
blocked-by-other-PR
|
215/5 |
Mathlib/ModelTheory/PartialEquiv.lean,Mathlib/ModelTheory/Substructures.lean |
2 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
225-47460 7 months ago |
225-47462 7 months ago |
0-668 11 minutes |
20248 |
peabrainiac author:peabrainiac |
feat(Topology/Compactness): first-countable locally path-connected spaces are delta-generated |
Shows that all first-countable locally path-connected spaces are delta-generated (so in particular all normed spaces and convex subsets thereof are), and that delta-generated spaces are equivalently generated by the unit interval or standard simplices.
---
- [ ] depends on: #21616
In principle, this should be close to all that's required to show that all simplicial complexes and CW-complexes are delta-generated; I just haven't done it yet because I'm not sure which file to best do it in.
[](https://gitpod.io/from-referrer/)
|
large-import
new-contributor
t-topology
merge-conflict
awaiting-author
blocked-by-other-PR
|
1189/813 |
Mathlib.lean,Mathlib/Geometry/Manifold/ChartedSpace.lean,Mathlib/Topology/Algebra/Module/LocallyConvex.lean,Mathlib/Topology/Compactness/DeltaGeneratedSpace.lean,Mathlib/Topology/Connected/LocPathConnected.lean,Mathlib/Topology/Connected/PathConnected.lean,Mathlib/Topology/ContinuousOn.lean,Mathlib/Topology/Homotopy/HSpaces.lean,Mathlib/Topology/Path.lean |
9 |
22 |
['YaelDillies', 'github-actions', 'kbuzzard', 'mathlib4-dependent-issues-bot', 'peabrainiac'] |
nobody |
215-39748 7 months ago |
215-39748 7 months ago |
39-21495 39 days |
20956 |
tomaz1502 author:tomaz1502 |
feat(Computability/QueryComplexity/Sort.lean): Formalization of upper bound of queries for merge sort |
This PR builds on top of #20924 to prove that merge sort (as defined in Lean's library) never executes more than `3 * n * ceil_log2 n` comparisons, where `n` is the size of the input list and `ceil_log2` is the ceil of the logarithm in base 2, which is defined in this PR.
Zulip discussion: https://leanprover.zulipchat.com/#narrow/channel/144837-PR-reviews/topic/.2318629.20runtime.20complexity.20of.20sorting.20a.20list
- [ ] depends on: #20924
Co-authored-by: Geoffrey Irving
---
[](https://gitpod.io/from-referrer/)
|
t-computability
blocked-by-other-PR
|
676/0 |
Mathlib.lean,Mathlib/Computability/QueryComplexity/Basic.lean,Mathlib/Computability/QueryComplexity/Defs.lean,Mathlib/Computability/QueryComplexity/Sort.lean |
4 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
204-52536 6 months ago |
233-66049 7 months ago |
0-41 41 seconds |
22233 |
pechersky author:pechersky |
feat(Algebra/Valued): `AdicExpansion.evalAt` |
---
- [ ] depends on: #22231
[](https://gitpod.io/from-referrer/)
|
t-topology
blocked-by-other-PR
|
488/0 |
Mathlib.lean,Mathlib/Topology/Algebra/Valued/AdicExpansion.lean |
2 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
201-27234 6 months ago |
201-27236 6 months ago |
0-412 6 minutes |
22232 |
pechersky author:pechersky |
feat(Algebra/Valued): `AdicExpansion.apprUpto` |
---
- [ ] depends on: #22231
[](https://gitpod.io/from-referrer/) |
t-topology
blocked-by-other-PR
|
399/0 |
Mathlib.lean,Mathlib/Topology/Algebra/Valued/AdicExpansion.lean |
2 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
201-27232 6 months ago |
201-27235 6 months ago |
0-414 6 minutes |
19372 |
Command-Master author:Command-Master |
find defeq abuse using diagnostics |
---
[](https://gitpod.io/from-referrer/)
- [ ] depends on: #19177 |
large-import
merge-conflict
blocked-by-other-PR
|
169/1 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter.lean,Mathlib/Tactic/Linter/FindDefEqAbuse.lean,MathlibTest/FindDefEqAbuse.lean,lakefile.lean |
6 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
193-83066 6 months ago |
193-83066 6 months ago |
0-0 0 seconds |
14060 |
YnirPaz author:YnirPaz |
feat(SetTheory/Ordinal/Clubs): define club sets and prove basic properties |
Create a file where club sets are defined and their basic properties are proven.
I also created a new recursion principle for ordinals, bounded recursion.
---
- [ ] depends on: #19189
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-logic
merge-conflict
blocked-by-other-PR
|
315/3 |
Mathlib.lean,Mathlib/Order/SuccPred/Limit.lean,Mathlib/SetTheory/Cardinal/Cofinality.lean,Mathlib/SetTheory/Ordinal/Arithmetic.lean,Mathlib/SetTheory/Ordinal/Club.lean,Mathlib/SetTheory/Ordinal/Topology.lean |
6 |
93 |
['YaelDillies', 'YnirPaz', 'alreadydone', 'dupuisf', 'github-actions', 'mathlib4-dependent-issues-bot', 'vihdzp', 'zeramorphic'] |
nobody |
193-24869 6 months ago |
193-24869 6 months ago |
92-44198 92 days |
17105 |
vihdzp author:vihdzp |
feat(Data/List/RunLength): run-length encoding |
We define the run-length encoding of a list. We provide a basic API, as well as a recursion principle.
---
- [ ] depends on: #16837
- [x] depends on: #17106
[](https://gitpod.io/from-referrer/)
|
t-data
merge-conflict
blocked-by-other-PR
|
286/1 |
Mathlib/Data/List/Flatten.lean,Mathlib/Data/List/RunLength.lean,Mathlib/Data/List/SplitBy.lean |
3 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
193-24622 6 months ago |
193-24622 6 months ago |
0-0 0 seconds |
16000 |
YaelDillies author:YaelDillies |
feat: Croot-Sisask Almost Periodicity |
Almost periodicity is nowadays a standard tool in additive combinatorics.
From LeanAPAP
---
- [ ] depends on: #15443
[](https://gitpod.io/from-referrer/)
|
t-analysis
t-combinatorics
blocked-by-other-PR
|
0/0 |
|
0 |
4 |
['github-actions', 'leanprover-community-mathlib4-bot', 'mergify'] |
nobody |
191-84856 6 months ago |
191-84861 6 months ago |
0-159 2 minutes |
22340 |
sinhp author:sinhp |
feat(CategoryTheory): Locally Cartesian Closed Categories (Beck-Chevalley Conditions) |
Building on top of the API of `ExponentiableMorphism` in #22321, we state and prove Beck-Chevalley conditions. This will be crucial for our development of polynomial functors along exponentiable morphisms.
Co-authored-by: Emily Riehl
---
- [ ] depends on: #22321
- [ ] depends on: #22319
- [ ] depends on: #21525
[](https://gitpod.io/from-referrer/)
|
large-import
t-category-theory
merge-conflict
blocked-by-other-PR
WIP
|
1144/24 |
Mathlib.lean,Mathlib/CategoryTheory/Comma/Over/Basic.lean,Mathlib/CategoryTheory/Comma/Over/Pullback.lean,Mathlib/CategoryTheory/Comma/Over/Sections.lean,Mathlib/CategoryTheory/Galois/Examples.lean,Mathlib/CategoryTheory/LocallyCartesianClosed/Basic.lean,Mathlib/CategoryTheory/LocallyCartesianClosed/BeckChevalley.lean,docs/references.bib |
8 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
191-72117 6 months ago |
191-72117 6 months ago |
0-17 17 seconds |
21275 |
joneugster author:joneugster |
feat(Cache): decompress downloaded files directly |
Extract downloaded files directly. This increases parallelism as files are downloaded in parallel and downloading/decompressing use different hardware (network/cpu)
---
- [ ] depends on: #21238
[](https://gitpod.io/from-referrer/)
|
CI
t-meta
merge-conflict
blocked-by-other-PR
WIP
|
66/15 |
Cache/IO.lean,Cache/Lean.lean,Cache/Requests.lean |
3 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
190-313 6 months ago |
190-313 6 months ago |
0-0 0 seconds |
20410 |
vihdzp author:vihdzp |
refactor: redefine `Equiv.Set.sumCompl = Equiv.sumCompl` |
It's still useful to have `Equiv.Set.sumCompl` around, as `simp` can't otherwise see through the def-eq `{x // x ∈ s} ⊕ {x // ¬ x ∈ s} = s ⊕ sᶜ`.
---
- [ ] depends on: #20850
[](https://gitpod.io/from-referrer/)
|
t-data
awaiting-CI
merge-conflict
blocked-by-other-PR
WIP
|
33/21 |
Mathlib/Logic/Equiv/Basic.lean,Mathlib/Logic/Equiv/Fintype.lean,Mathlib/Logic/Equiv/Set.lean |
3 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
177-19794 5 months ago |
177-19794 5 months ago |
0-0 0 seconds |
23145 |
joneugster author:joneugster |
feat(CategoryTheory/Enriched/Limits): add IsConicalLimits |
---
- [ ] depends on: #23142
[](https://gitpod.io/from-referrer/)
|
infinity-cosmos
t-category-theory
merge-conflict
blocked-by-other-PR
|
221/9 |
Mathlib.lean,Mathlib/CategoryTheory/Enriched/Limits/HasConicalLimits.lean,Mathlib/CategoryTheory/Enriched/Limits/IsConicalLimit.lean |
3 |
3 |
['github-actions', 'joelriou', 'mathlib4-dependent-issues-bot'] |
nobody |
175-59172 5 months ago |
175-59172 5 months ago |
0-806 13 minutes |
20222 |
eric-wieser author:eric-wieser |
feat: generalize lemmas about derivatives |
Rather than creating a huge diff by shuffling things around, this generalizes everything in-place and swaps between `section`s for topological and normed vector spaces.
The rationale for this approach is that:
* we may further generalize the results of this file, and this avoids us jumbling up the order multiple times unnecessarily.
* this greatly reduces the chance of merge conflicts
---
- [ ] depends on: #21065
[](https://gitpod.io/from-referrer/)
|
t-analysis
merge-conflict
blocked-by-other-PR
|
554/50 |
Mathlib/Analysis/Calculus/Deriv/Basic.lean,Mathlib/Analysis/Calculus/FDeriv/Basic.lean,MathlibTest/Recall.lean |
3 |
8 |
['adomani', 'eric-wieser', 'github-actions', 'leanprover-bot', 'mathlib4-dependent-issues-bot'] |
nobody |
166-5217 5 months ago |
166-5217 5 months ago |
16-16341 16 days |
21769 |
JovanGerb author:JovanGerb |
feat: extensible `push_neg` tactic |
This was started by point (3) of https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Possible.20improvements.20to.20Lean.2FMathlib/near/499085779
To be able to use `push_neg` more generally, this PR reimplements the tactic so that it is extensible. So, users can tag lemmas to be used by `push_neg`.
This PR tags lemmas concerning empty/nonempty, subsingleton/nontrivial, and finite/infinite to be used in `push_neg`.
Additionally, the tactic is extended to be able to push any constant that you want to push, and `push_neg` is now a macro for `push Not`. So far, I've tried to add lemmas for pushing `Real.log`. I could imagine it could also be used for `Real.exp`, `pow`, `mul`, `smul`, or even `Set.mem`. (the `Set.mem` lemmas are mostly tagged with `@[simp]` already, but `push_mem` could be more readable than `simp` or `dsimp`). Or a combination of pushing `Not` and `Set.compl` could be useful.
The implementation is with the `simp` infrastructure, but instead of using post lemmas, like in `simp`, `push` uses `pre` lemmas, so we rewrite each expression before its subterms are rewritten. This is a more efficient way to "push" constants recursively. Most lemmas are added via the `@[push]` attribute, but a few cases require some special handling, so they are implemented "by hand" in a simproc that is tried after the `push` lemmas.
For example the simproc simplifies `¬∀ n, p` ⇨ `∃ n, ¬p`, but, this is overridden by the `push` lemma that rewrites `¬(p → q)` ⇨ `p ∧ ¬q` (which doesn't apply at every forall)
---
- [ ] depends on: #21965
[](https://gitpod.io/from-referrer/)
|
large-import
t-meta
merge-conflict
blocked-by-other-PR
|
786/544 |
Archive/Imo/Imo1988Q6.lean,Archive/Imo/Imo2013Q5.lean,Archive/Imo/Imo2024Q3.lean,Archive/ZagierTwoSquares.lean,Counterexamples/Phillips.lean,Mathlib.lean,Mathlib/Algebra/BigOperators/Finprod.lean,Mathlib/Algebra/BigOperators/Group/Finset/Defs.lean,Mathlib/Algebra/CharP/MixedCharZero.lean,Mathlib/Algebra/Group/Action/Defs.lean,Mathlib/Algebra/Group/Basic.lean,Mathlib/Algebra/Group/Defs.lean,Mathlib/Algebra/Group/Pi/Basic.lean,Mathlib/Algebra/Group/Pointwise/Finset/Basic.lean,Mathlib/Algebra/GroupWithZero/Action/Defs.lean,Mathlib/Algebra/Lie/Submodule.lean,Mathlib/Algebra/Lie/Weights/Linear.lean,Mathlib/Algebra/Module/DedekindDomain.lean,Mathlib/Algebra/Order/Antidiag/Nat.lean,Mathlib/Algebra/Order/Archimedean/IndicatorCard.lean,Mathlib/Algebra/Order/GroupWithZero/Canonical.lean,Mathlib/Algebra/Order/Monoid/Canonical/Defs.lean,Mathlib/Algebra/Polynomial/Degree/Definitions.lean,Mathlib/Algebra/Ring/Commute.lean,Mathlib/Algebra/Ring/Defs.lean,Mathlib/AlgebraicTopology/DoldKan/Degeneracies.lean,Mathlib/Analysis/Analytic/OfScalars.lean,Mathlib/Analysis/Analytic/Order.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Order.lean,Mathlib/Analysis/Calculus/FDeriv/Norm.lean,Mathlib/Analysis/Complex/OpenMapping.lean,Mathlib/Analysis/Complex/Polynomial/UnitTrinomial.lean,Mathlib/Analysis/SpecialFunctions/Log/Basic.lean,Mathlib/Analysis/SpecialFunctions/MulExpNegMulSqIntegral.lean,Mathlib/Combinatorics/Enumerative/Composition.lean,Mathlib/Combinatorics/Enumerative/DyckWord.lean,Mathlib/Combinatorics/SimpleGraph/Acyclic.lean,Mathlib/Combinatorics/SimpleGraph/Diam.lean,Mathlib/Combinatorics/SimpleGraph/Path.lean,Mathlib/Combinatorics/SimpleGraph/Turan.lean,Mathlib/Computability/AkraBazzi/GrowsPolynomially.lean,Mathlib/Data/Analysis/Filter.lean,Mathlib/Data/ENat/Lattice.lean,Mathlib/Data/Finite/Defs.lean,Mathlib/Data/Finset/Card.lean,Mathlib/Data/Finset/Empty.lean,Mathlib/Data/Finset/Powerset.lean,Mathlib/Data/Finset/SDiff.lean,Mathlib/Data/Fintype/Basic.lean,Mathlib/Data/Fintype/Card.lean,Mathlib/Data/Fintype/Prod.lean,Mathlib/Data/Fintype/Sum.lean,Mathlib/Data/Nat/Defs.lean,Mathlib/Data/Nat/Factorization/PrimePow.lean,Mathlib/Data/Nat/Lattice.lean,Mathlib/Data/Nat/Order/Lemmas.lean,Mathlib/Data/Nat/PrimeFin.lean,Mathlib/Data/Ordmap/Ordset.lean,Mathlib/Data/Real/Archimedean.lean,Mathlib/Data/Set/Basic.lean,Mathlib/Data/Set/Insert.lean,Mathlib/Data/Set/Lattice.lean,Mathlib/Data/Set/Operations.lean,Mathlib/Data/ZMod/Basic.lean,Mathlib/Dynamics/OmegaLimit.lean,Mathlib/FieldTheory/JacobsonNoether.lean,Mathlib/Geometry/Manifold/ChartedSpace.lean,Mathlib/Geometry/Manifold/PartitionOfUnity.lean,Mathlib/GroupTheory/ArchimedeanDensely.lean,Mathlib/GroupTheory/OrderOfElement.lean,Mathlib/GroupTheory/Perm/ClosureSwap.lean,Mathlib/GroupTheory/SpecificGroups/Cyclic.lean,Mathlib/GroupTheory/SpecificGroups/ZGroup.lean,Mathlib/InformationTheory/Hamming.lean,Mathlib/LinearAlgebra/AffineSpace/AffineSubspace.lean,Mathlib/LinearAlgebra/Eigenspace/Zero.lean,Mathlib/LinearAlgebra/Matrix/SemiringInverse.lean,Mathlib/LinearAlgebra/Multilinear/Basic.lean,Mathlib/LinearAlgebra/Reflection.lean,Mathlib/Logic/IsEmpty.lean,Mathlib/Logic/Nontrivial/Defs.lean,Mathlib/MeasureTheory/Covering/Differentiation.lean,Mathlib/MeasureTheory/Decomposition/Lebesgue.lean,Mathlib/MeasureTheory/Function/ConvergenceInMeasure.lean,Mathlib/MeasureTheory/Function/UniformIntegrable.lean,Mathlib/MeasureTheory/Group/FundamentalDomain.lean,Mathlib/MeasureTheory/Integral/Bochner.lean,Mathlib/MeasureTheory/Integral/Lebesgue.lean,Mathlib/MeasureTheory/Measure/DiracProba.lean,Mathlib/MeasureTheory/Measure/Haar/NormedSpace.lean,Mathlib/MeasureTheory/Measure/MeasureSpace.lean,Mathlib/MeasureTheory/Measure/MeasureSpaceDef.lean,Mathlib/MeasureTheory/Measure/OpenPos.lean,Mathlib/MeasureTheory/Measure/Typeclasses.lean,Mathlib/MeasureTheory/OuterMeasure/Basic.lean,Mathlib/MeasureTheory/SetAlgebra.lean,Mathlib/ModelTheory/Ultraproducts.lean,Mathlib/NumberTheory/AbelSummation.lean,Mathlib/NumberTheory/ArithmeticFunction.lean,Mathlib/NumberTheory/Divisors.lean |
149 |
4 |
['adomani', 'github-actions', 'grunweg', 'mathlib4-dependent-issues-bot'] |
nobody |
160-49182 5 months ago |
160-49184 5 months ago |
5-54179 5 days |
22321 |
sinhp author:sinhp |
feat(CategoryTheory): Locally Cartesian Closed Categories (Definition) |
This PR defines locally cartesian closed categories in terms of existence of the pushforward functors (right adjoint to the pullback functor) for all morphisms. We develop basic API and prove the following:
1. Existence of the pushforward functors is equivalent to cartesian closed slices.
2. Any locally cartesian closed category with a terminal object is cartesian closed.
3. The slices of a locally cartesian closed category are locally cartesian closed.
Some of the content is based on the project of formalization of polynomial functors at the Trimester "Prospect of Formal Mathematics" at the Hausdorff Institute (HIM) in Bonn. https://github.com/sinhp/Poly
I found this implementation of locally cartesian closed categories amenable to polynomial functors formalization.
Co-authored-by: Emily Riehl
---
- [ ] depends on: #21525
- [ ] depends on: #22319
[](https://gitpod.io/from-referrer/)
|
large-import
t-category-theory
merge-conflict
blocked-by-other-PR
|
812/24 |
Mathlib.lean,Mathlib/CategoryTheory/Comma/Over/Basic.lean,Mathlib/CategoryTheory/Comma/Over/Pullback.lean,Mathlib/CategoryTheory/Comma/Over/Sections.lean,Mathlib/CategoryTheory/Galois/Examples.lean,Mathlib/CategoryTheory/LocallyCartesianClosed/Basic.lean |
6 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
156-76332 5 months ago |
156-76333 5 months ago |
0-336 5 minutes |
22319 |
sinhp author:sinhp |
feat(CategoryTheory): Locally Cartesian Closed Categories (Sections Right Adjoint) |
we define the `Over.sections` functor in the file `CategoryTheory.Comma.Over.Sections` and prove that it is a right adjoint to the `Over.star`, thereby solving an existing TODO in `Over.pullback` file.
The `sections` functor is used to define the right adjoint to the pullback functor `Over.pullback` in the development of LCCCs. Moreover, the rest of added lemmas and theorems to `CategoryTheory.Comma.Over.Pullback` are crucial for the development of LCCCs in the next PR.
---
- [ ] depends on: #21525
[](https://gitpod.io/from-referrer/)
|
large-import
t-category-theory
merge-conflict
blocked-by-other-PR
|
547/24 |
Mathlib.lean,Mathlib/CategoryTheory/Comma/Over/Basic.lean,Mathlib/CategoryTheory/Comma/Over/Pullback.lean,Mathlib/CategoryTheory/Comma/Over/Sections.lean,Mathlib/CategoryTheory/Galois/Examples.lean |
5 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
156-76332 5 months ago |
156-76334 5 months ago |
0-2084 34 minutes |
19475 |
YaelDillies author:YaelDillies |
feat: group markings |
From LeanCamCombi
---
- [ ] depends on: #21342
[](https://gitpod.io/from-referrer/)
|
t-algebra
blocked-by-other-PR
WIP
label:t-algebra$ |
196/12 |
Mathlib.lean,Mathlib/Geometry/Group/Marking.lean,Mathlib/Topology/Algebra/ConstMulAction.lean,Mathlib/Topology/Algebra/Group/Quotient.lean |
4 |
12 |
['YaelDillies', 'b-mehta', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
155-11463 5 months ago |
155-11482 5 months ago |
22-16818 22 days |
24010 |
grunweg author:grunweg |
feat(Counterexamples): a non-negative function, not a.e. zero, with vanishing lowe… |
…r Lebesgue integral.
Came up in #23707, let's document this while we're at it.
---
- [ ] depends on: #20722
[](https://gitpod.io/from-referrer/)
|
t-measure-probability
please-adopt
blocked-by-other-PR
WIP
|
110/0 |
Counterexamples.lean,Counterexamples/LIntegralZero.lean |
2 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
152-51678 4 months ago |
152-51680 4 months ago |
0-22 22 seconds |
24040 |
FR-vdash-bot author:FR-vdash-bot |
refactor: unbundle algebra from `(NonUnital){Seminormed, Normed}(Comm)Ring` |
---
- [ ] depends on: #23966
[](https://gitpod.io/from-referrer/)
|
slow-typeclass-synthesis
t-algebra
t-analysis
merge-conflict
blocked-by-other-PR
label:t-algebra$ |
3775/3674 |
Archive/Imo/Imo1998Q2.lean,Counterexamples/LinearOrderWithPosMulPosEqZero.lean,Mathlib/Algebra/Algebra/RestrictScalars.lean,Mathlib/Algebra/Module/ZLattice/Basic.lean,Mathlib/Algebra/Module/ZLattice/Covolume.lean,Mathlib/Algebra/Order/Field/Canonical.lean,Mathlib/Algebra/Order/Field/Rat.lean,Mathlib/Algebra/Order/Floor/Ring.lean,Mathlib/Algebra/Order/GroupWithZero/Canonical.lean,Mathlib/Algebra/Order/GroupWithZero/Finset.lean,Mathlib/Algebra/Order/Hom/Monoid.lean,Mathlib/Algebra/Order/Nonneg/Field.lean,Mathlib/Algebra/Order/Nonneg/Ring.lean,Mathlib/Algebra/Order/Ring/Nat.lean,Mathlib/Analysis/Analytic/Basic.lean,Mathlib/Analysis/Analytic/CPolynomial.lean,Mathlib/Analysis/Analytic/CPolynomialDef.lean,Mathlib/Analysis/Analytic/ChangeOrigin.lean,Mathlib/Analysis/Analytic/Composition.lean,Mathlib/Analysis/Analytic/Constructions.lean,Mathlib/Analysis/Analytic/Inverse.lean,Mathlib/Analysis/Analytic/IsolatedZeros.lean,Mathlib/Analysis/Analytic/IteratedFDeriv.lean,Mathlib/Analysis/Analytic/Linear.lean,Mathlib/Analysis/Analytic/OfScalars.lean,Mathlib/Analysis/Analytic/Order.lean,Mathlib/Analysis/Analytic/Polynomial.lean,Mathlib/Analysis/Analytic/RadiusLiminf.lean,Mathlib/Analysis/Analytic/Uniqueness.lean,Mathlib/Analysis/Analytic/Within.lean,Mathlib/Analysis/Asymptotics/AsymptoticEquivalent.lean,Mathlib/Analysis/Asymptotics/Defs.lean,Mathlib/Analysis/Asymptotics/Lemmas.lean,Mathlib/Analysis/Asymptotics/SpecificAsymptotics.lean,Mathlib/Analysis/Asymptotics/TVS.lean,Mathlib/Analysis/Asymptotics/Theta.lean,Mathlib/Analysis/BoundedVariation.lean,Mathlib/Analysis/BoxIntegral/Basic.lean,Mathlib/Analysis/BoxIntegral/DivergenceTheorem.lean,Mathlib/Analysis/BoxIntegral/Integrability.lean,Mathlib/Analysis/BoxIntegral/Partition/Additive.lean,Mathlib/Analysis/BoxIntegral/Partition/Measure.lean,Mathlib/Analysis/CStarAlgebra/Basic.lean,Mathlib/Analysis/CStarAlgebra/CStarMatrix.lean,Mathlib/Analysis/CStarAlgebra/Classes.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Basic.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Instances.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Integral.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Isometric.lean,Mathlib/Analysis/CStarAlgebra/ContinuousLinearMap.lean,Mathlib/Analysis/CStarAlgebra/ContinuousMap.lean,Mathlib/Analysis/CStarAlgebra/Exponential.lean,Mathlib/Analysis/CStarAlgebra/GelfandDuality.lean,Mathlib/Analysis/CStarAlgebra/Matrix.lean,Mathlib/Analysis/CStarAlgebra/Module/Constructions.lean,Mathlib/Analysis/CStarAlgebra/Module/Defs.lean,Mathlib/Analysis/CStarAlgebra/Multiplier.lean,Mathlib/Analysis/CStarAlgebra/Spectrum.lean,Mathlib/Analysis/CStarAlgebra/Unitization.lean,Mathlib/Analysis/CStarAlgebra/lpSpace.lean,Mathlib/Analysis/Calculus/AddTorsor/AffineMap.lean,Mathlib/Analysis/Calculus/AddTorsor/Coord.lean,Mathlib/Analysis/Calculus/BumpFunction/Basic.lean,Mathlib/Analysis/Calculus/BumpFunction/Convolution.lean,Mathlib/Analysis/Calculus/BumpFunction/FiniteDimension.lean,Mathlib/Analysis/Calculus/BumpFunction/InnerProduct.lean,Mathlib/Analysis/Calculus/BumpFunction/Normed.lean,Mathlib/Analysis/Calculus/Conformal/InnerProduct.lean,Mathlib/Analysis/Calculus/Conformal/NormedSpace.lean,Mathlib/Analysis/Calculus/ContDiff/Basic.lean,Mathlib/Analysis/Calculus/ContDiff/Bounds.lean,Mathlib/Analysis/Calculus/ContDiff/CPolynomial.lean,Mathlib/Analysis/Calculus/ContDiff/Defs.lean,Mathlib/Analysis/Calculus/ContDiff/FTaylorSeries.lean,Mathlib/Analysis/Calculus/ContDiff/FaaDiBruno.lean,Mathlib/Analysis/Calculus/ContDiff/FiniteDimension.lean,Mathlib/Analysis/Calculus/ContDiff/Operations.lean,Mathlib/Analysis/Calculus/ContDiff/RCLike.lean,Mathlib/Analysis/Calculus/ContDiff/WithLp.lean,Mathlib/Analysis/Calculus/DSlope.lean,Mathlib/Analysis/Calculus/Deriv/Abs.lean,Mathlib/Analysis/Calculus/Deriv/Add.lean,Mathlib/Analysis/Calculus/Deriv/AffineMap.lean,Mathlib/Analysis/Calculus/Deriv/Basic.lean,Mathlib/Analysis/Calculus/Deriv/Comp.lean,Mathlib/Analysis/Calculus/Deriv/Inv.lean,Mathlib/Analysis/Calculus/Deriv/Inverse.lean,Mathlib/Analysis/Calculus/Deriv/Linear.lean,Mathlib/Analysis/Calculus/Deriv/Mul.lean,Mathlib/Analysis/Calculus/Deriv/Prod.lean,Mathlib/Analysis/Calculus/Deriv/Shift.lean,Mathlib/Analysis/Calculus/Deriv/Slope.lean,Mathlib/Analysis/Calculus/Deriv/Star.lean,Mathlib/Analysis/Calculus/Deriv/Support.lean,Mathlib/Analysis/Calculus/Deriv/ZPow.lean,Mathlib/Analysis/Calculus/DiffContOnCl.lean,Mathlib/Analysis/Calculus/FDeriv/Add.lean,Mathlib/Analysis/Calculus/FDeriv/Analytic.lean,Mathlib/Analysis/Calculus/FDeriv/Basic.lean,Mathlib/Analysis/Calculus/FDeriv/Bilinear.lean |
630 |
n/a |
['FR-vdash-bot', 'github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
151-70292 4 months ago |
unknown |
unknown |
24058 |
FR-vdash-bot author:FR-vdash-bot |
refactor: unbundle algebra from `*NormedField` |
---
- [ ] depends on: #24040
[](https://gitpod.io/from-referrer/)
|
slow-typeclass-synthesis
t-algebra
t-analysis
merge-conflict
blocked-by-other-PR
label:t-algebra$ |
4602/4346 |
Archive/Hairer.lean,Archive/Imo/Imo1998Q2.lean,Counterexamples/LinearOrderWithPosMulPosEqZero.lean,Mathlib/Algebra/Algebra/RestrictScalars.lean,Mathlib/Algebra/Module/ZLattice/Basic.lean,Mathlib/Algebra/Module/ZLattice/Covolume.lean,Mathlib/Algebra/Order/Field/Canonical.lean,Mathlib/Algebra/Order/Field/Rat.lean,Mathlib/Algebra/Order/Floor/Ring.lean,Mathlib/Algebra/Order/GroupWithZero/Canonical.lean,Mathlib/Algebra/Order/GroupWithZero/Finset.lean,Mathlib/Algebra/Order/Hom/Monoid.lean,Mathlib/Algebra/Order/Nonneg/Field.lean,Mathlib/Algebra/Order/Nonneg/Ring.lean,Mathlib/Algebra/Order/Ring/Nat.lean,Mathlib/Analysis/Analytic/Basic.lean,Mathlib/Analysis/Analytic/CPolynomial.lean,Mathlib/Analysis/Analytic/CPolynomialDef.lean,Mathlib/Analysis/Analytic/ChangeOrigin.lean,Mathlib/Analysis/Analytic/Composition.lean,Mathlib/Analysis/Analytic/Constructions.lean,Mathlib/Analysis/Analytic/Inverse.lean,Mathlib/Analysis/Analytic/IsolatedZeros.lean,Mathlib/Analysis/Analytic/IteratedFDeriv.lean,Mathlib/Analysis/Analytic/Linear.lean,Mathlib/Analysis/Analytic/OfScalars.lean,Mathlib/Analysis/Analytic/Order.lean,Mathlib/Analysis/Analytic/Polynomial.lean,Mathlib/Analysis/Analytic/RadiusLiminf.lean,Mathlib/Analysis/Analytic/Uniqueness.lean,Mathlib/Analysis/Analytic/Within.lean,Mathlib/Analysis/Asymptotics/AsymptoticEquivalent.lean,Mathlib/Analysis/Asymptotics/Defs.lean,Mathlib/Analysis/Asymptotics/Lemmas.lean,Mathlib/Analysis/Asymptotics/SpecificAsymptotics.lean,Mathlib/Analysis/Asymptotics/SuperpolynomialDecay.lean,Mathlib/Analysis/Asymptotics/TVS.lean,Mathlib/Analysis/Asymptotics/Theta.lean,Mathlib/Analysis/BoundedVariation.lean,Mathlib/Analysis/BoxIntegral/Basic.lean,Mathlib/Analysis/BoxIntegral/DivergenceTheorem.lean,Mathlib/Analysis/BoxIntegral/Integrability.lean,Mathlib/Analysis/BoxIntegral/Partition/Additive.lean,Mathlib/Analysis/BoxIntegral/Partition/Measure.lean,Mathlib/Analysis/CStarAlgebra/Basic.lean,Mathlib/Analysis/CStarAlgebra/CStarMatrix.lean,Mathlib/Analysis/CStarAlgebra/Classes.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Basic.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Instances.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Integral.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Isometric.lean,Mathlib/Analysis/CStarAlgebra/ContinuousLinearMap.lean,Mathlib/Analysis/CStarAlgebra/ContinuousMap.lean,Mathlib/Analysis/CStarAlgebra/Exponential.lean,Mathlib/Analysis/CStarAlgebra/GelfandDuality.lean,Mathlib/Analysis/CStarAlgebra/Matrix.lean,Mathlib/Analysis/CStarAlgebra/Module/Constructions.lean,Mathlib/Analysis/CStarAlgebra/Module/Defs.lean,Mathlib/Analysis/CStarAlgebra/Multiplier.lean,Mathlib/Analysis/CStarAlgebra/Spectrum.lean,Mathlib/Analysis/CStarAlgebra/Unitization.lean,Mathlib/Analysis/CStarAlgebra/lpSpace.lean,Mathlib/Analysis/Calculus/AddTorsor/AffineMap.lean,Mathlib/Analysis/Calculus/AddTorsor/Coord.lean,Mathlib/Analysis/Calculus/BumpFunction/Basic.lean,Mathlib/Analysis/Calculus/BumpFunction/Convolution.lean,Mathlib/Analysis/Calculus/BumpFunction/FiniteDimension.lean,Mathlib/Analysis/Calculus/BumpFunction/InnerProduct.lean,Mathlib/Analysis/Calculus/BumpFunction/Normed.lean,Mathlib/Analysis/Calculus/Conformal/InnerProduct.lean,Mathlib/Analysis/Calculus/Conformal/NormedSpace.lean,Mathlib/Analysis/Calculus/ContDiff/Basic.lean,Mathlib/Analysis/Calculus/ContDiff/Bounds.lean,Mathlib/Analysis/Calculus/ContDiff/CPolynomial.lean,Mathlib/Analysis/Calculus/ContDiff/Defs.lean,Mathlib/Analysis/Calculus/ContDiff/FTaylorSeries.lean,Mathlib/Analysis/Calculus/ContDiff/FaaDiBruno.lean,Mathlib/Analysis/Calculus/ContDiff/FiniteDimension.lean,Mathlib/Analysis/Calculus/ContDiff/Operations.lean,Mathlib/Analysis/Calculus/ContDiff/RCLike.lean,Mathlib/Analysis/Calculus/ContDiff/WithLp.lean,Mathlib/Analysis/Calculus/DSlope.lean,Mathlib/Analysis/Calculus/Deriv/Abs.lean,Mathlib/Analysis/Calculus/Deriv/Add.lean,Mathlib/Analysis/Calculus/Deriv/AffineMap.lean,Mathlib/Analysis/Calculus/Deriv/Basic.lean,Mathlib/Analysis/Calculus/Deriv/Comp.lean,Mathlib/Analysis/Calculus/Deriv/Inv.lean,Mathlib/Analysis/Calculus/Deriv/Inverse.lean,Mathlib/Analysis/Calculus/Deriv/Linear.lean,Mathlib/Analysis/Calculus/Deriv/Mul.lean,Mathlib/Analysis/Calculus/Deriv/Pi.lean,Mathlib/Analysis/Calculus/Deriv/Polynomial.lean,Mathlib/Analysis/Calculus/Deriv/Pow.lean,Mathlib/Analysis/Calculus/Deriv/Prod.lean,Mathlib/Analysis/Calculus/Deriv/Shift.lean,Mathlib/Analysis/Calculus/Deriv/Slope.lean,Mathlib/Analysis/Calculus/Deriv/Star.lean,Mathlib/Analysis/Calculus/Deriv/Support.lean,Mathlib/Analysis/Calculus/Deriv/ZPow.lean |
665 |
7 |
['FR-vdash-bot', 'github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
150-65083 4 months ago |
151-40902 4 months ago* |
0-0 0 seconds* |
24106 |
FR-vdash-bot author:FR-vdash-bot |
refactor: unbundle algebra from `*CStarAlgebra` |
---
[](https://gitpod.io/from-referrer/)
- [ ] depends on: #24058
|
slow-typeclass-synthesis
t-algebra
t-analysis
merge-conflict
blocked-by-other-PR
label:t-algebra$ |
4702/4459 |
Archive/Hairer.lean,Archive/Imo/Imo1998Q2.lean,Counterexamples/LinearOrderWithPosMulPosEqZero.lean,Mathlib/Algebra/Algebra/RestrictScalars.lean,Mathlib/Algebra/Module/ZLattice/Basic.lean,Mathlib/Algebra/Module/ZLattice/Covolume.lean,Mathlib/Algebra/Order/Field/Canonical.lean,Mathlib/Algebra/Order/Field/Rat.lean,Mathlib/Algebra/Order/Floor/Ring.lean,Mathlib/Algebra/Order/GroupWithZero/Canonical.lean,Mathlib/Algebra/Order/GroupWithZero/Finset.lean,Mathlib/Algebra/Order/Hom/Monoid.lean,Mathlib/Algebra/Order/Nonneg/Field.lean,Mathlib/Algebra/Order/Nonneg/Ring.lean,Mathlib/Algebra/Order/Ring/Nat.lean,Mathlib/Analysis/Analytic/Basic.lean,Mathlib/Analysis/Analytic/CPolynomial.lean,Mathlib/Analysis/Analytic/CPolynomialDef.lean,Mathlib/Analysis/Analytic/ChangeOrigin.lean,Mathlib/Analysis/Analytic/Composition.lean,Mathlib/Analysis/Analytic/Constructions.lean,Mathlib/Analysis/Analytic/Inverse.lean,Mathlib/Analysis/Analytic/IsolatedZeros.lean,Mathlib/Analysis/Analytic/IteratedFDeriv.lean,Mathlib/Analysis/Analytic/Linear.lean,Mathlib/Analysis/Analytic/OfScalars.lean,Mathlib/Analysis/Analytic/Order.lean,Mathlib/Analysis/Analytic/Polynomial.lean,Mathlib/Analysis/Analytic/RadiusLiminf.lean,Mathlib/Analysis/Analytic/Uniqueness.lean,Mathlib/Analysis/Analytic/Within.lean,Mathlib/Analysis/Asymptotics/AsymptoticEquivalent.lean,Mathlib/Analysis/Asymptotics/Defs.lean,Mathlib/Analysis/Asymptotics/Lemmas.lean,Mathlib/Analysis/Asymptotics/SpecificAsymptotics.lean,Mathlib/Analysis/Asymptotics/SuperpolynomialDecay.lean,Mathlib/Analysis/Asymptotics/TVS.lean,Mathlib/Analysis/Asymptotics/Theta.lean,Mathlib/Analysis/BoundedVariation.lean,Mathlib/Analysis/BoxIntegral/Basic.lean,Mathlib/Analysis/BoxIntegral/DivergenceTheorem.lean,Mathlib/Analysis/BoxIntegral/Integrability.lean,Mathlib/Analysis/BoxIntegral/Partition/Additive.lean,Mathlib/Analysis/BoxIntegral/Partition/Measure.lean,Mathlib/Analysis/CStarAlgebra/ApproximateUnit.lean,Mathlib/Analysis/CStarAlgebra/Basic.lean,Mathlib/Analysis/CStarAlgebra/CStarMatrix.lean,Mathlib/Analysis/CStarAlgebra/Classes.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Basic.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Instances.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Integral.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Isometric.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Order.lean,Mathlib/Analysis/CStarAlgebra/ContinuousLinearMap.lean,Mathlib/Analysis/CStarAlgebra/ContinuousMap.lean,Mathlib/Analysis/CStarAlgebra/Exponential.lean,Mathlib/Analysis/CStarAlgebra/GelfandDuality.lean,Mathlib/Analysis/CStarAlgebra/Hom.lean,Mathlib/Analysis/CStarAlgebra/Matrix.lean,Mathlib/Analysis/CStarAlgebra/Module/Constructions.lean,Mathlib/Analysis/CStarAlgebra/Module/Defs.lean,Mathlib/Analysis/CStarAlgebra/Multiplier.lean,Mathlib/Analysis/CStarAlgebra/PositiveLinearMap.lean,Mathlib/Analysis/CStarAlgebra/SpecialFunctions/PosPart.lean,Mathlib/Analysis/CStarAlgebra/Spectrum.lean,Mathlib/Analysis/CStarAlgebra/Unitization.lean,Mathlib/Analysis/CStarAlgebra/lpSpace.lean,Mathlib/Analysis/Calculus/AddTorsor/AffineMap.lean,Mathlib/Analysis/Calculus/AddTorsor/Coord.lean,Mathlib/Analysis/Calculus/BumpFunction/Basic.lean,Mathlib/Analysis/Calculus/BumpFunction/Convolution.lean,Mathlib/Analysis/Calculus/BumpFunction/FiniteDimension.lean,Mathlib/Analysis/Calculus/BumpFunction/InnerProduct.lean,Mathlib/Analysis/Calculus/BumpFunction/Normed.lean,Mathlib/Analysis/Calculus/Conformal/InnerProduct.lean,Mathlib/Analysis/Calculus/Conformal/NormedSpace.lean,Mathlib/Analysis/Calculus/ContDiff/Basic.lean,Mathlib/Analysis/Calculus/ContDiff/Bounds.lean,Mathlib/Analysis/Calculus/ContDiff/CPolynomial.lean,Mathlib/Analysis/Calculus/ContDiff/Defs.lean,Mathlib/Analysis/Calculus/ContDiff/FTaylorSeries.lean,Mathlib/Analysis/Calculus/ContDiff/FaaDiBruno.lean,Mathlib/Analysis/Calculus/ContDiff/FiniteDimension.lean,Mathlib/Analysis/Calculus/ContDiff/Operations.lean,Mathlib/Analysis/Calculus/ContDiff/RCLike.lean,Mathlib/Analysis/Calculus/ContDiff/WithLp.lean,Mathlib/Analysis/Calculus/DSlope.lean,Mathlib/Analysis/Calculus/Deriv/Abs.lean,Mathlib/Analysis/Calculus/Deriv/Add.lean,Mathlib/Analysis/Calculus/Deriv/AffineMap.lean,Mathlib/Analysis/Calculus/Deriv/Basic.lean,Mathlib/Analysis/Calculus/Deriv/Comp.lean,Mathlib/Analysis/Calculus/Deriv/Inv.lean,Mathlib/Analysis/Calculus/Deriv/Inverse.lean,Mathlib/Analysis/Calculus/Deriv/Linear.lean,Mathlib/Analysis/Calculus/Deriv/Mul.lean,Mathlib/Analysis/Calculus/Deriv/Pi.lean,Mathlib/Analysis/Calculus/Deriv/Polynomial.lean,Mathlib/Analysis/Calculus/Deriv/Pow.lean,Mathlib/Analysis/Calculus/Deriv/Prod.lean |
670 |
5 |
['FR-vdash-bot', 'github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
150-18224 4 months ago |
150-20531 4 months ago* |
0-0 0 seconds* |
24016 |
plp127 author:plp127 |
feat: fine uniformity |
Adds the fine uniformity, and proves some properties.
---
- [ ] depends on: #24096 for showing the induced topology is equal on completely regular spaces
[](https://gitpod.io/from-referrer/)
|
t-topology
blocked-by-other-PR
|
283/0 |
Mathlib.lean,Mathlib/Topology/UniformSpace/FineUniformity.lean,Mathlib/Topology/UniformSpace/Uniformizable.lean |
3 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
149-37909 4 months ago |
149-37911 4 months ago |
2-85349 2 days |
21238 |
joneugster author:joneugster |
feat(Cache): enable partial cache in downstream projects |
Add features to `cache` and cleanup code:
* enable partial cache retrieval in downstream projects: `lake exe cache get MyProject.Basic` downloads only the relevant cache to build `MyProject/Basic.lean`
* accept paths `Mathlib/Init.lean` and modules `Mathlib.Init` likewise
#21822
* accept folders in the form `Mathlib/Data` or `Mathlib.Data` and does a directory walk to find all`.lean` files therein
#21838
* throw error if sources contain a build loop.
#21632
* cleanup
* internally cache now works with the module names as keys (used paths before)
#21834
* eliminate need of parsing the `lake_manifest.json`, use the Lean search path from `LEAN_SRC_PATH` instead.
#21666
* eliminate most hard-coded file paths, generating them from the module name with `Lean.findLean`
#21818
* add documentation
---
- [x] depends on: #21834
- [ ] depends on: #21838
### Follow-up PR:
- #21842
### Notes:
- replaces: #21195
- should address: #8767
- should address: #20568
### Completed:
- [x] depends on: #21632
- [x] ~~depends on: #21663~~
- [x] depends on: #21666
- [x] depends on: #21701
- [x] depends on: #21703
- [x] depends on: #21704
- [x] depends on: #21705
- [x] depends on: #21707
- [x] depends on: #21711
- [x] depends on: #21750
- [x] depends on: #21815
- [x] depends on: #21816
- [x] depends on: #21817
- [x] depends on: #21818
- [x] depends on: #21822
- [x] depends on: #21830
- #21848
[](https://gitpod.io/from-referrer/)
|
CI
t-meta
merge-conflict
blocked-by-other-PR
|
231/118 |
Cache/Hashing.lean,Cache/IO.lean,Cache/Main.lean |
3 |
n/a |
['github-actions', 'grunweg', 'joneugster', 'kim-em', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
148-56737 4 months ago |
unknown |
unknown |
21842 |
joneugster author:joneugster |
refactor(Cache): use module name for file hash instead of non-resolved file path |
This invalidates cache once, similarly to when the `lean-toolchain` gets bumped or the `lakefile` modified.
---
- [ ] depends on: #21238
[](https://gitpod.io/from-referrer/)
|
CI
t-meta
merge-conflict
blocked-by-other-PR
|
284/139 |
Cache/Hashing.lean,Cache/IO.lean,Cache/Lean.lean,Cache/Main.lean |
4 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
148-56613 4 months ago |
211-53636 6 months ago* |
0-0 0 seconds* |
19467 |
quangvdao author:quangvdao |
feat(MvPolynomial/Equiv): Add `MvPolynomial.finSuccEquivNth` |
This PR adds `MvPolynomial.finSuccEquivNth`, which is the algebra isomorphism between `MvPolynomial (Fin (n + 1)) R` and `Polynomial (MvPolynomial (Fin n) R)` by identifying the `p`-th variable as the indeterminate.
This generalizes `MvPolynomial.finSuccEquiv` which is only for the `0`-th variable. The supporting theorems for the `Nth` version are identical to the current version, with the `Nth` version deduced from the former.
These changes require new definitions in `Finsupp/Fin`, which is a separate PR.
Co-authored-by: Yaël Dillies ---
- [ ] depends on: #19315
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
blocked-by-other-PR
label:t-algebra$ |
541/163 |
Mathlib/Algebra/BigOperators/Fin.lean,Mathlib/Algebra/BigOperators/Finsupp.lean,Mathlib/Algebra/MvPolynomial/Equiv.lean,Mathlib/Data/Fin/Basic.lean,Mathlib/Data/Fin/Tuple/Basic.lean,Mathlib/Data/Finsupp/Fin.lean,scripts/nolints_prime_decls.txt |
7 |
9 |
['acmepjz', 'github-actions', 'grunweg', 'mathlib4-dependent-issues-bot', 'quangvdao'] |
nobody |
148-50834 4 months ago |
148-50834 4 months ago |
0-790 13 minutes |
22547 |
joelriou author:joelriou |
feat(CategoryTheory/Abelian): construction of reduced left resolutions |
The standard functorial free resolution of a `R`-module `M` does not directly extend to free resolutions of (bounded above) complexes because the free `R`-module functor does preserve zero morphisms. In this PR, we provide a general construction which takes functorial left resolutions and modify them by considering a suitable direct factor so that it preserves zero morphisms.
---
- [ ] depends on: #22539
[](https://gitpod.io/from-referrer/)
|
t-category-theory
blocked-by-other-PR
WIP
|
514/19 |
Mathlib.lean,Mathlib/Algebra/Homology/HomologicalComplex.lean,Mathlib/Algebra/Homology/LeftResolutions/Basic.lean,Mathlib/Algebra/Homology/LeftResolutions/Reduced.lean,Mathlib/Algebra/Homology/LeftResolutions/Transport.lean,Mathlib/CategoryTheory/Limits/Shapes/Kernels.lean |
6 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
138-55145 4 months ago |
192-77460 6 months ago |
0-358 5 minutes |
22556 |
joelriou author:joelriou |
feat(Algebra/Category/ModuleCat): a functorial projective resolution |
---
- [ ] depends on: #22539
[](https://gitpod.io/from-referrer/)
|
t-category-theory
blocked-by-other-PR
|
315/19 |
Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/LeftResolutions.lean,Mathlib/Algebra/Homology/HomologicalComplex.lean,Mathlib/Algebra/Homology/LeftResolutions/Basic.lean,Mathlib/CategoryTheory/Limits/Shapes/Kernels.lean |
5 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
138-55015 4 months ago |
192-71773 6 months ago |
0-516 8 minutes |
24549 |
grunweg author:grunweg |
feat: define embedded submanifolds, attempt 1 |
Not meant to be merged (I think a different design is better); opening this so I can find this more easily.
---
- [ ] depends on: #23040
[](https://gitpod.io/from-referrer/)
|
t-differential-geometry
merge-conflict
blocked-by-other-PR
WIP
|
1445/2 |
Mathlib.lean,Mathlib/Analysis/NormedSpace/HahnBanach/Splits.lean,Mathlib/Geometry/Manifold/Diffeomorph.lean,Mathlib/Geometry/Manifold/EmbeddedSubmanifold.lean,Mathlib/Geometry/Manifold/IsImmersionEmbedding.lean,Mathlib/Geometry/Manifold/LocalDiffeomorph.lean,Mathlib/Geometry/Manifold/MSplits.lean,Mathlib/LinearAlgebra/Prod.lean |
8 |
2 |
['leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
133-11702 4 months ago |
133-11702 4 months ago |
0-1 1 second |
11003 |
thorimur author:thorimur |
chore: migrate to `tfae` block tactic |
Migrates to the `tfae` block tactic syntax, eliminating uses of `tfae_have` and `tfae_finish`.
---
- [ ] depends on: #11000
- [ ] depends on: #10991
[](https://gitpod.io/from-referrer/)
|
t-meta
merge-conflict
blocked-by-other-PR
WIP
|
1267/1081 |
Mathlib/Algebra/Exact.lean,Mathlib/Algebra/Homology/ShortComplex/ExactFunctor.lean,Mathlib/Algebra/Order/ToIntervalMod.lean,Mathlib/Analysis/BoxIntegral/Box/Basic.lean,Mathlib/Analysis/InnerProductSpace/Basic.lean,Mathlib/Analysis/LocallyConvex/WithSeminorms.lean,Mathlib/Analysis/NormedSpace/OperatorNorm/NormedSpace.lean,Mathlib/Analysis/RCLike/Basic.lean,Mathlib/Analysis/SpecificLimits/Normed.lean,Mathlib/CategoryTheory/Abelian/Exact.lean,Mathlib/CategoryTheory/Bicategory/Kan/Adjunction.lean,Mathlib/FieldTheory/Galois.lean,Mathlib/FieldTheory/KummerExtension.lean,Mathlib/GroupTheory/Nilpotent.lean,Mathlib/LinearAlgebra/Eigenspace/Zero.lean,Mathlib/MeasureTheory/Group/Action.lean,Mathlib/NumberTheory/FLT/Basic.lean,Mathlib/Order/CompactlyGenerated/Basic.lean,Mathlib/Order/Height.lean,Mathlib/Order/WellFoundedSet.lean,Mathlib/RingTheory/Bezout.lean,Mathlib/RingTheory/DiscreteValuationRing/TFAE.lean,Mathlib/RingTheory/Flat/EquationalCriterion.lean,Mathlib/RingTheory/Henselian.lean,Mathlib/RingTheory/LocalRing/RingHom/Basic.lean,Mathlib/RingTheory/Valuation/Basic.lean,Mathlib/RingTheory/Valuation/ValuationRing.lean,Mathlib/SetTheory/Ordinal/Topology.lean,Mathlib/Tactic/TFAE.lean,Mathlib/Topology/Algebra/Group/SubmonoidClosure.lean,Mathlib/Topology/Category/CompHaus/EffectiveEpi.lean,Mathlib/Topology/Category/Profinite/EffectiveEpi.lean,Mathlib/Topology/Category/Stonean/EffectiveEpi.lean,Mathlib/Topology/Inseparable.lean,Mathlib/Topology/LocallyClosed.lean,Mathlib/Topology/LocallyConstant/Basic.lean,Mathlib/Topology/NoetherianSpace.lean,Mathlib/Topology/Order/LeftRightNhds.lean,Mathlib/Topology/Separation.lean,Mathlib/Topology/UniformSpace/UniformConvergence.lean,scripts/noshake.json,test/tfae.lean |
42 |
2 |
['github-actions', 'leanprover-community-mathlib4-bot'] |
nobody |
133-10518 4 months ago |
133-10518 4 months ago |
0-0 0 seconds |
16186 |
joneugster author:joneugster |
chore: use emoji-variant-selector `\uFE0F` for emojis ✅️,❌️,💥️,🟡️ |
Append the emoji-variant selector `\uFE0F` to these 4 unicode symbols which should always be rendered as emojis.
---
This has been done in core, so it makes sense to do the same in Mathlib.
- [x] depends on: leanprover/lean4#5173
- [ ] depends on: #16215
[](https://gitpod.io/from-referrer/)
|
t-linter
merge-conflict
awaiting-author
blocked-by-other-PR
|
28/28 |
.github/workflows/lean4checker.yml,.github/workflows/nightly_detect_failure.yml,.github/workflows/update_dependencies_zulip.yml,scripts/lean-pr-testing-comments.sh,test/AssertExists.lean |
5 |
3 |
['github-actions', 'leanprover-community-mathlib4-bot', 'urkud'] |
nobody |
133-10202 4 months ago |
133-10202 4 months ago |
7-61243 7 days |
21853 |
smmercuri author:smmercuri |
feat: the adele ring of a number field is locally compact |
---
- [ ] depends on: #21158
- [ ] depends on: #21847
[](https://gitpod.io/from-referrer/)
|
large-import
t-number-theory
merge-conflict
blocked-by-other-PR
WIP
|
398/3 |
Mathlib.lean,Mathlib/Algebra/Order/GroupWithZero/Canonical.lean,Mathlib/NumberTheory/NumberField/AdeleRing.lean,Mathlib/RingTheory/DedekindDomain/AdicValuation.lean,Mathlib/RingTheory/DedekindDomain/FiniteAdeleRing.lean,Mathlib/RingTheory/Ideal/Quotient/Basic.lean,Mathlib/Topology/Algebra/Group/Basic.lean,Mathlib/Topology/Algebra/Valued/LocallyCompact.lean,Mathlib/Topology/Algebra/Valued/WithZeroMulInt.lean |
9 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
130-62339 4 months ago |
133-11340 4 months ago |
0-0 0 seconds |
15654 |
TpmKranz author:TpmKranz |
feat(Computability): language-preserving maps between NFA and RE |
Map REs to NFAs via Thompson's construction and NFAs to REs using GNFAs
Last chunk of #12648
---
- [ ] depends on: #15651
- [ ] depends on: #15649
[](https://gitpod.io/from-referrer/)
|
awaiting-zulip
t-computability
new-contributor
merge-conflict
blocked-by-other-PR
|
985/2 |
Mathlib.lean,Mathlib/Computability/GNFA.lean,Mathlib/Computability/Language.lean,Mathlib/Computability/NFA.lean,Mathlib/Computability/RegularExpressions.lean,Mathlib/Data/FinEnum/Option.lean,docs/references.bib |
7 |
3 |
['github-actions', 'leanprover-community-mathlib4-bot', 'meithecatte'] |
nobody |
130-44037 4 months ago |
130-44042 4 months ago |
0-179 2 minutes |
16553 |
grunweg author:grunweg |
WIP: tinkering with orientable manifolds |
- wait for Rida's PR to get merged
- PR the "normed space" part separately
- WIP: a linear isomorphism on a connected set is either orientation-preserving or orientation-preserving: this will require #8738, it seems
- [ ] depends on: #16239
- [ ] depends on: #8738
---
[](https://gitpod.io/from-referrer/)
|
t-differential-geometry
blocked-by-other-PR
WIP
|
287/0 |
Mathlib.lean,Mathlib/Geometry/Manifold/Instances/Sphere.lean,Mathlib/Geometry/Manifold/Orientable.lean |
3 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
127-47215 4 months ago |
366-10080 1 year ago |
0-0 0 seconds |
24550 |
grunweg author:grunweg |
feat: define `SliceModel` typeclass for models with corners for embedded submanifolds |
Still work in progress: TODO write a proper module doc-string and commit message.
---
- [ ] depends on: #23040 (at least morally)
[](https://gitpod.io/from-referrer/)
|
t-differential-geometry
merge-conflict
blocked-by-other-PR
WIP
|
1214/0 |
Mathlib.lean,Mathlib/Analysis/NormedSpace/HahnBanach/Splits.lean,Mathlib/Geometry/Manifold/IsImmersionEmbedding.lean,Mathlib/Geometry/Manifold/LocalDiffeomorph.lean,Mathlib/Geometry/Manifold/MSplits.lean,Mathlib/Geometry/Manifold/SliceModel.lean |
6 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
127-41300 4 months ago |
127-41732 4 months ago |
0-0 0 seconds |
18755 |
FR-vdash-bot author:FR-vdash-bot |
refactor: deprecate `LinearIsometryClass` |
---
- [ ] depends on: #18748
- [ ] depends on: #18754
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-analysis
merge-conflict
blocked-by-other-PR
label:t-algebra$ |
243/116 |
Mathlib/Analysis/CStarAlgebra/Spectrum.lean,Mathlib/Analysis/LocallyConvex/WeakOperatorTopology.lean,Mathlib/Analysis/Normed/Algebra/Spectrum.lean,Mathlib/Analysis/Normed/Group/Uniform.lean,Mathlib/Analysis/Normed/Operator/LinearIsometry.lean,Mathlib/Topology/Algebra/Module/Basic.lean,Mathlib/Topology/Algebra/Module/CharacterSpace.lean,Mathlib/Topology/Algebra/Module/FiniteDimension.lean,Mathlib/Topology/Algebra/Module/StrongTopology.lean,Mathlib/Topology/Algebra/Module/WeakDual.lean,Mathlib/Topology/Homeomorph.lean,Mathlib/Topology/MetricSpace/Isometry.lean,scripts/no_lints_prime_decls.txt |
13 |
5 |
['FR-vdash-bot', 'github-actions', 'leanprover-bot', 'mathlib4-dependent-issues-bot'] |
nobody |
126-50746 4 months ago |
302-7007 9 months ago |
0-602 10 minutes |
5863 |
eric-wieser author:eric-wieser |
feat: add elaborators for concrete matrices |
---
- [x] depends on: #5866
- [ ] depends on: #5897
[](https://gitpod.io/from-referrer/)
|
t-meta
blocked-by-other-PR
help-wanted
|
257/7 |
Mathlib/Control/Monad/Cont.lean,Mathlib/Data/Matrix/Auto.lean,MathlibTest/matrix_auto.lean |
3 |
7 |
['eric-wieser', 'github-actions', 'kim-em', 'leanprover-community-bot-assistant'] |
nobody |
111-45541 3 months ago |
111-45562 3 months ago |
0-0 0 seconds |
25141 |
eric-wieser author:eric-wieser |
feat: basis for multilinear maps |
This attempts to tease an intermediate result out of #11155, which lets us show that multilinear maps are free even if their codomain is not finite.
I guess this continues from https://github.com/leanprover-community/mathlib3/pull/10504 and https://github.com/leanprover-community/mathlib3/pull/14199.
---
- [ ] depends on: #11155
- [ ] depends on: #25142
- [ ] depends on: #25169
- [ ] depends on: #25166
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebra
merge-conflict
blocked-by-other-PR
label:t-algebra$ |
507/45 |
Mathlib.lean,Mathlib/LinearAlgebra/DFinsupp.lean,Mathlib/LinearAlgebra/DFinsupp/PiTensorProduct.lean,Mathlib/LinearAlgebra/DirectSum/Finsupp.lean,Mathlib/LinearAlgebra/DirectSum/PiTensorProduct.lean,Mathlib/LinearAlgebra/Multilinear/Basic.lean,Mathlib/LinearAlgebra/Multilinear/Basis.lean,Mathlib/LinearAlgebra/Multilinear/DFinsupp.lean,Mathlib/LinearAlgebra/Multilinear/DirectSum.lean,Mathlib/LinearAlgebra/Multilinear/FiniteDimensional.lean,Mathlib/LinearAlgebra/Multilinear/Pi.lean |
11 |
4 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
106-65344 3 months ago |
106-65345 3 months ago |
0-0 0 seconds |
25750 |
robin-carlier author:robin-carlier |
feat(Tactic/CategoryTheory): bicategory extension for `rotate_isos` |
This PR registers some lemmas to the `rotate_isos` tactic so that it applies in bicategorical contexts.
For instance, if `α : g ⟶ h` is an invertible 2-cells, the term `f ◁ α ` is also recognized as invertible, with inverse `f ◁ α' `, where `α'` is the expression for the inverse constructed by the tactic.
Without this extension, the tactic would only construct the generic `inv (f ◁ α)` as inverse for this term.
---
- [ ] depends on: #25747
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #24633.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/24633* |
t-category-theory
t-meta
blocked-by-other-PR
|
1206/0 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/CategoryTheory/RotateIsos/Bicategory.lean,Mathlib/Tactic/CategoryTheory/RotateIsos/Cancelable.lean,Mathlib/Tactic/CategoryTheory/RotateIsos/Core.lean,Mathlib/Tactic/CategoryTheory/RotateIsos/Lemmas.lean,MathlibTest/CategoryTheory/RotateIsos.lean,scripts/noshake.json |
8 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
93-8414 3 months ago |
93-8583 3 months ago |
0-0 0 seconds |
25748 |
robin-carlier author:robin-carlier |
feat(Tactic/CategoryTheory): Initial lemmas for the `rotate_iso` tactic |
This PR records an initial set of lemmas to be used by the WIP `rotate_isos` tactic.
---
- [ ] depends on: #25746
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #24506.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/24506* |
t-meta
blocked-by-other-PR
|
496/0 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/CategoryTheory/RotateIsos/Cancelable.lean,Mathlib/Tactic/CategoryTheory/RotateIsos/Lemmas.lean,scripts/noshake.json |
5 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
93-8413 3 months ago |
93-8414 3 months ago |
0-0 0 seconds |
25747 |
robin-carlier author:robin-carlier |
feat(Tactic/CategoryTheory): the `rotate_isos` tactic |
We define a `rotate_isos` tactic for category theory in mathlib.
At its core, the tactic transform terms of type `α(1) ≫ ⋯ ≫ α(k) = β(1) ≫ ⋯ ≫ β(l)` where `α` and `β` are families of morphisms in whith the first `i` morphisms of the left-hand side and the last `j` morphisms of the right-hand side are isomorhisms, into terms of type `α(k-i) ≫ ⋯ ≫ α(k) ≫ inv β(l) ≫ ⋯ ≫ β(l-j+1) = inv α(j) ≫ ⋯ ≫ inv α(1) ≫⋯ ≫ β(l-j)`.
The construction of the inverses of expression are caried at the `Expr` levels are built out of the expressions of the morphisms, for instance, for this tactic, the inverse of `F.map (G.map (H.map f.hom)))` will directly be `F.map (G.map (H.map f.inv)))` (which would have to be re-simplified), rather than an `inv` term form an `IsIso` instance.
The tactic can be applied at a local hypothesis or at the main goal, or can be used through a `rotate_isos%` term elaborator if e.g one wants to add such a "rotated" form to a `simp` or `rw` call.
We also support removing morphisms "from the right" of the lhs, rather than from the right.
---
The motivations behind this tactic are the following :
- This tactic can "autogenerate" lemmas and terms generalizing lemmas such as [CategoryTheory.Iso.hom_inv_id_app_app_app](https://leanprover-community.github.io/mathlib4_docs/Mathlib/CategoryTheory/NatIso.html#CategoryTheory.Iso.hom_inv_id_app_app_app). This can also generate lemmas `F.map (G.map f.hom) ≫F.map (G.map f.inv) = 𝟙 _`, and can be used to unlock a `simp` call that blocks at an expression of the form `F.map (G.map f.hom) ≫F.map (G.map f.inv) `.
- Currently, cancelling morphisms "from the right" in an expression in category theory is a bit of a pain. You have to first reassociate the expression, perform multiple calls to `Iso.inv_comp_eq`, reassociate, etc. This at least automates this process in a fairly straightforward way.
- There are expressions in category theory that have no "right forms", e.g the pentagon axiom for monoidal categories, which has many variations in the way one can read the diagram of isomorphisms that represents it. Elaborators such as `rotate_iso%` easily generates all possible forms of such identities from one single form, and avoids having to state multiple forms of the same equality as individual lemmas.
- I have been playing with medium-sized diagrams of isomorphisms recently (think for example vertical/horizontal compositions of `CatCommSq`, whiskering a corner of such diagrams, etc.), and it made me wish a lot of time that such easy way to transforms equalities to equivalent forms were available.
- [ ] depends on: #25746
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #24454.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/24454* |
t-category-theory
t-meta
awaiting-author
blocked-by-other-PR
WIP
|
871/0 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/CategoryTheory/RotateIsos/Cancelable.lean,Mathlib/Tactic/CategoryTheory/RotateIsos/Core.lean,Mathlib/Tactic/CategoryTheory/RotateIsos/Lemmas.lean,MathlibTest/CategoryTheory/RotateIsos.lean,scripts/noshake.json |
7 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
93-8413 3 months ago |
93-8666 3 months ago |
0-0 0 seconds |
25751 |
robin-carlier author:robin-carlier |
feat(Tactic/CategoryTheory): monoidal extension of `rotate_isos` |
This PR registers some lemmas to the `rotate_isos` tactic so that it applies in monoidal contexts.
For instance, if α : y ⟶ z is an invertible morphism, the term x ◁ α is also recognized as invertible, with inverse x ◁ α' , where α' is the expression for the inverse constructed by the tactic.
Without this extension, the tactic would only construct the generic inv (x ◁ α) as inverse for this term.
We also take care of terms of the form `f ⊗ g`
---
- [ ] depends on: #25747
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #24634.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/24634* |
t-category-theory
t-meta
blocked-by-other-PR
|
1362/0 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/CategoryTheory/RotateIsos/Cancelable.lean,Mathlib/Tactic/CategoryTheory/RotateIsos/Core.lean,Mathlib/Tactic/CategoryTheory/RotateIsos/Lemmas.lean,Mathlib/Tactic/CategoryTheory/RotateIsos/Monoidal.lean,MathlibTest/CategoryTheory/RotateIsos.lean,scripts/noshake.json |
8 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
93-7432 3 months ago |
93-8278 3 months ago |
0-0 0 seconds |
25752 |
robin-carlier author:robin-carlier |
feat(Tactic/CategoryTheory): whiskering lemmas for `rotate_isos` |
This PR extends the base set of terms recognized by the `rotate_isos` tactic to include terms of the form `whiskerLeft F f`, `isoWhiskerLeft F e`, and `NatTrans.hcomp`/ `NatIso.hcomp`.
---
- [ ] depends on: #25747
Technically, it could depend solely on #24506, but there’s not much point getting this merged if the base tactic is not there.
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #24650.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/24650* |
t-meta
blocked-by-other-PR
|
1365/0 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/CategoryTheory/RotateIsos/Cancelable.lean,Mathlib/Tactic/CategoryTheory/RotateIsos/Core.lean,Mathlib/Tactic/CategoryTheory/RotateIsos/Lemmas.lean,MathlibTest/CategoryTheory/RotateIsos.lean,scripts/noshake.json |
7 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
93-7433 3 months ago |
93-7434 3 months ago |
0-0 0 seconds |
25912 |
BoltonBailey author:BoltonBailey |
feat: add simp lemmas for trig functions on `π * 2⁻¹` |
This PR adds a number of simp lemmas to reduce trig functions evaluated on `π * 2⁻¹`. This allows `simp` to reduce expressions such as `sin (π * (1 / 2))`
---
- [ ] depends on: #25911 [experiment with simp normal form]
Original PR: #24213 |
t-analysis
awaiting-author
blocked-by-other-PR
|
45/0 |
Mathlib/Analysis/SpecialFunctions/Trigonometric/Basic.lean |
1 |
3 |
['BoltonBailey', 'github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
89-68925 2 months ago |
89-69521 2 months ago |
0-136 2 minutes |
26108 |
xroblot author:xroblot |
feat(NumberField/IsCM): compute the index of the subgroup of real units |
This PR continues the work from #23694.
---
- [ ] depends on: #26107
|
large-import
t-number-theory
blocked-by-other-PR
|
443/75 |
Mathlib/Algebra/Field/Equiv.lean,Mathlib/Algebra/Group/Invertible/Basic.lean,Mathlib/AlgebraicGeometry/Morphisms/Proper.lean,Mathlib/FieldTheory/LinearDisjoint.lean,Mathlib/GroupTheory/GroupAction/FixedPoints.lean,Mathlib/LinearAlgebra/Dimension/Localization.lean,Mathlib/NumberTheory/NumberField/CMField.Lean,Mathlib/NumberTheory/NumberField/Units/Basic.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 |
15 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'xroblot'] |
nobody |
86-69643 2 months ago |
86-69644 2 months ago |
0-875 14 minutes |
24434 |
joelriou author:joelriou |
feat(CategoryTheory): effectiveness of descent |
Co-authored-by: Christian Merten [christian@merten.dev](mailto:christian@merten.dev)
---
- [ ] depends on: #24411
- [x] depends on: #24382
- [ ] depends on: #25971
- [x] depends on: #13539
[](https://gitpod.io/from-referrer/)
|
t-category-theory
merge-conflict
blocked-by-other-PR
WIP
|
4052/66 |
Mathlib.lean,Mathlib/CategoryTheory/Bicategory/Adjunction/Adj.lean,Mathlib/CategoryTheory/Bicategory/Adjunction/BaseChange.lean,Mathlib/CategoryTheory/Bicategory/Adjunction/Basic.lean,Mathlib/CategoryTheory/Bicategory/Adjunction/Mate.lean,Mathlib/CategoryTheory/Bicategory/Functor/Cat.lean,Mathlib/CategoryTheory/Bicategory/Functor/LocallyDiscrete.lean,Mathlib/CategoryTheory/Bicategory/Functor/Strict.lean,Mathlib/CategoryTheory/Bicategory/Opposite.lean,Mathlib/CategoryTheory/CommSq.lean,Mathlib/CategoryTheory/Limits/Shapes/Pullback/CommSq.lean,Mathlib/CategoryTheory/Sites/Descent/DescentData.lean,Mathlib/CategoryTheory/Sites/Descent/DescentDataAsCoalgebra.lean,Mathlib/CategoryTheory/Sites/Descent/DescentDataDoublePrime.lean,Mathlib/CategoryTheory/Sites/Descent/DescentDataPrime.lean,Mathlib/CategoryTheory/Sites/Descent/IsPrestack.lean,Mathlib/CategoryTheory/Sites/Descent/IsStack.lean,Mathlib/CategoryTheory/Sites/Descent/ModuleCat.lean,Mathlib/CategoryTheory/Sites/Descent/PullbackStruct.lean |
19 |
n/a |
['callesonne', 'chrisflav', 'github-actions', 'joelriou', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
86-65798 2 months ago |
unknown |
unknown |
18771 |
joelriou author:joelriou |
feat(LinearAlgebra/ExteriorPower): exterior powers of free modules are free |
Co-authored-by: sophie.morel@ens-lyon.fr
---
- [ ] depends on: #18662
- [x] depends on: #18534
- [x] depends on: #18651
- [x] depends on: #18590
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
blocked-by-other-PR
WIP
label:t-algebra$ |
1185/160 |
Mathlib.lean,Mathlib/Analysis/NormedSpace/Multilinear/Curry.lean,Mathlib/Analysis/NormedSpace/PiTensorProduct/ProjectiveSeminorm.lean,Mathlib/Data/Sum/Basic.lean,Mathlib/LinearAlgebra/ExteriorPower/Basic.lean,Mathlib/LinearAlgebra/ExteriorPower/Basis.lean,Mathlib/LinearAlgebra/ExteriorPower/Generators.lean,Mathlib/LinearAlgebra/ExteriorPower/Pairing.lean,Mathlib/LinearAlgebra/Multilinear/Basic.lean,Mathlib/LinearAlgebra/Multilinear/TensorProduct.lean,Mathlib/LinearAlgebra/PiTensorProduct/Basic.lean,Mathlib/LinearAlgebra/PiTensorProduct/Finite.lean,Mathlib/LinearAlgebra/PiTensorProduct/Generators.lean,Mathlib/LinearAlgebra/Span.lean,Mathlib/LinearAlgebra/TensorAlgebra/ToTensorPower.lean,Mathlib/LinearAlgebra/TensorPower/Basic.lean,Mathlib/LinearAlgebra/TensorPower/Pairing.lean,Mathlib/Logic/Function/Basic.lean,Mathlib/RingTheory/PiTensorProduct.lean |
19 |
3 |
['alreadydone', 'github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
86-4680 2 months ago |
302-7006 9 months ago |
0-0 0 seconds |
25926 |
BoltonBailey author:BoltonBailey |
feat: add lemma about `degreeOf_eq_degree` |
Adds MvPolynomial.degreeOf_eq_degree, which states that the degree of a particular variable in a multivariate polynomial is equal to the degree of the single-variable polynomial obtained by treating the multivariable polynomial as a single variable polynomial over multivariable polynomials in the remaining variables.
This PR continues the work from #12664.
- [ ] depends on: #25920
depends on https://github.com/leanprover-community/mathlib4/pull/25920 |
t-algebra
blocked-by-other-PR
label:t-algebra$ |
50/0 |
Mathlib/Algebra/MvPolynomial/Equiv.lean |
1 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
84-65035 2 months ago |
84-65036 2 months ago |
5-1720 5 days |
25925 |
BoltonBailey author:BoltonBailey |
feat: file for lemmas about MvPolynomials over NoZeroDivisors |
This PR continues the work from #11106 and #11073
Original PR: https://github.com/leanprover-community/mathlib4/pull/11106
- [x] depends on: #11095
- [x] depends on: #11094
- [ ] depends on: #25926 [We need this lemma to establish fact about degreeOf n (p + q)]
|
t-algebra
blocked-by-other-PR
label:t-algebra$ |
85/0 |
Mathlib/Algebra/MvPolynomial/NoZeroDivisors.lean |
1 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
83-43636 2 months ago |
83-43637 2 months ago |
0-0 0 seconds |
20051 |
Timeroot author:Timeroot |
feat: `Clone` and some instances |
Defines clones (`Clone`). And there is a file, `Instances.lean`, that gives several most important examples of Clones. In particular, it has all of the clones (in an appropriately general form) that occur in [Post's Lattice](https://en.wikipedia.org/wiki/Post%27s_lattice), and [later proving](https://github.com/leanprover-community/mathlib4/pull/24744) the completeness of Post's Lattice is why I'm making this PR.
(Edit: Used to also say "Defined operads (`Operad`), symmetric operads (`SymmOperad`), and clones ... There is a proof that all clones have a natural operad structure.". This has been scrapped.)
---
- [x] depends on: #20133 [basics and notations]
- [x] depends on: #20134 [permutations]
- [x] depends on: #20138 [operad]
- [x] depends on: #20141 [clone]
- [x] depends on: #23459 [defs]
- [ ] depends on: #23460 [basic]
[](https://gitpod.io/from-referrer/)
|
t-algebra
awaiting-author
blocked-by-other-PR
label:t-algebra$ |
623/0 |
Mathlib.lean,Mathlib/Algebra/Clone/Basic.lean,Mathlib/Algebra/Clone/Defs.lean,Mathlib/Algebra/Clone/Instances.lean,Mathlib/Data/Fin/Basic.lean |
5 |
32 |
['Timeroot', 'YaelDillies', 'eric-wieser', 'github-actions', 'jcommelin', 'kbuzzard', 'kim-em', 'mathlib4-dependent-issues-bot', 'wmacmil'] |
nobody |
81-26905 2 months ago |
166-54545 5 months ago |
43-16103 43 days |
26391 |
grunweg author:grunweg |
feat: immersed submanifolds |
Still under construction
---
- [ ] depends on: #26087
- [ ] depends on: #23040
Better version of #24549.
[](https://gitpod.io/from-referrer/)
|
t-differential-geometry
blocked-by-other-PR
WIP
|
1418/0 |
Mathlib.lean,Mathlib/Analysis/NormedSpace/HahnBanach/Splits.lean,Mathlib/Geometry/Manifold/EmbeddedSubmanifold.lean,Mathlib/Geometry/Manifold/IsImmersionEmbedding.lean,Mathlib/Geometry/Manifold/MSplits.lean |
5 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
79-57464 2 months ago |
80-23371 2 months ago |
0-0 0 seconds |
18662 |
joelriou author:joelriou |
feat(LinearAlgebra/ExteriorPower): generators of the exterior powers |
---
- [x] depends on: #18534
- [x] depends on: #18590
- [ ] depends on: #26464
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
blocked-by-other-PR
WIP
label:t-algebra$ |
818/158 |
Mathlib.lean,Mathlib/Analysis/NormedSpace/Multilinear/Curry.lean,Mathlib/Analysis/NormedSpace/PiTensorProduct/ProjectiveSeminorm.lean,Mathlib/Data/Sum/Basic.lean,Mathlib/LinearAlgebra/ExteriorPower/Basic.lean,Mathlib/LinearAlgebra/ExteriorPower/Generators.lean,Mathlib/LinearAlgebra/Multilinear/Basic.lean,Mathlib/LinearAlgebra/Multilinear/TensorProduct.lean,Mathlib/LinearAlgebra/PiTensorProduct/Basic.lean,Mathlib/LinearAlgebra/PiTensorProduct/Finite.lean,Mathlib/LinearAlgebra/PiTensorProduct/Generators.lean,Mathlib/LinearAlgebra/Span.lean,Mathlib/LinearAlgebra/TensorPower.lean,Mathlib/Logic/Function/Basic.lean,Mathlib/RingTheory/PiTensorProduct.lean |
15 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
78-11135 2 months ago |
302-7010 9 months ago |
0-0 0 seconds |
18735 |
joelriou author:joelriou |
feat(Algebra/Module): presentation of the exterior power |
Given a presentation of a `R`-module `M`, we obtain a presentation of `⋀[R]^n M`.
---
(Still one sorry left.)
- [ ] depends on: #18527
- [ ] depends on: #18432
- [ ] depends on: #26464
- [ ] depends on: #18534
- [ ] depends on: #18662
- [x] depends on: #18590
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
blocked-by-other-PR
WIP
label:t-algebra$ |
1856/157 |
Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/ExteriorPower.lean,Mathlib/Algebra/Module/Presentation/Basic.lean,Mathlib/Algebra/Module/Presentation/ExteriorPower.lean,Mathlib/Algebra/Module/Presentation/PiTensor.lean,Mathlib/Algebra/Module/Presentation/Tensor.lean,Mathlib/Analysis/NormedSpace/Multilinear/Curry.lean,Mathlib/Analysis/NormedSpace/PiTensorProduct/ProjectiveSeminorm.lean,Mathlib/Data/Sum/Basic.lean,Mathlib/LinearAlgebra/ExteriorPower/Basic.lean,Mathlib/LinearAlgebra/ExteriorPower/Generators.lean,Mathlib/LinearAlgebra/Multilinear/Basic.lean,Mathlib/LinearAlgebra/Multilinear/TensorProduct.lean,Mathlib/LinearAlgebra/PiTensorProduct/Basic.lean,Mathlib/LinearAlgebra/PiTensorProduct/Finite.lean,Mathlib/LinearAlgebra/PiTensorProduct/Generators.lean,Mathlib/LinearAlgebra/Span.lean,Mathlib/LinearAlgebra/TensorPower.lean,Mathlib/Logic/Function/Basic.lean,Mathlib/RingTheory/PiTensorProduct.lean |
20 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
78-7109 2 months ago |
302-7008 9 months ago |
0-0 0 seconds |
18551 |
joelriou author:joelriou |
feat(AlgebraicGeometry): the algebraic De Rham complex |
If `B` is an `A`-algebra, we construct the algebraic De Rham complex of `B` over `A`: it is a cochain complex of `A`-modules.
---
- [ ] depends on: #18735
- [ ] depends on: #18662
- [ ] depends on: #26464
- [ ] depends on: #18534
- [ ] depends on: #18527
- [x] depends on: #18440
- [ ] depends on: #18432
- [x] depends on: #18408
- [x] depends on: #18389
- [x] depends on: #18374
- [x] depends on: #18359
- [x] depends on: #18332
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-algebraic-geometry
merge-conflict
blocked-by-other-PR
WIP
label:t-algebra$ |
2836/156 |
Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/ExteriorPower.lean,Mathlib/Algebra/Module/Presentation/Basic.lean,Mathlib/Algebra/Module/Presentation/Cokernel.lean,Mathlib/Algebra/Module/Presentation/Differentials.lean,Mathlib/Algebra/Module/Presentation/DirectSum.lean,Mathlib/Algebra/Module/Presentation/ExteriorPower.lean,Mathlib/Algebra/Module/Presentation/PiTensor.lean,Mathlib/Algebra/Module/Presentation/RestrictScalars.lean,Mathlib/Algebra/Module/Presentation/Tensor.lean,Mathlib/Analysis/NormedSpace/Multilinear/Curry.lean,Mathlib/Analysis/NormedSpace/PiTensorProduct/ProjectiveSeminorm.lean,Mathlib/Data/Finsupp/Defs.lean,Mathlib/Data/Sum/Basic.lean,Mathlib/LinearAlgebra/ExteriorPower/Basic.lean,Mathlib/LinearAlgebra/ExteriorPower/Generators.lean,Mathlib/LinearAlgebra/Multilinear/Basic.lean,Mathlib/LinearAlgebra/Multilinear/TensorProduct.lean,Mathlib/LinearAlgebra/PiTensorProduct/Basic.lean,Mathlib/LinearAlgebra/PiTensorProduct/Finite.lean,Mathlib/LinearAlgebra/PiTensorProduct/Generators.lean,Mathlib/LinearAlgebra/Span.lean,Mathlib/LinearAlgebra/TensorPower.lean,Mathlib/Logic/Function/Basic.lean,Mathlib/RingTheory/DeRham/Basic.lean,Mathlib/RingTheory/PiTensorProduct.lean |
26 |
n/a |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
78-7105 2 months ago |
unknown |
unknown |
24411 |
joelriou author:joelriou |
feat(CategoryTheory): descent of morphisms for a pseudofunctor |
Let `C` be a category and `F : Pseudofunctor (LocallyDiscrete Cᵒᵖ) Cat`. Given `S : C`, and objects `M` and `N` in `F.obj (.mk (op S))`, we define a presheaf of types `F.presheafHom M N` on the category `Over S`: its sections on a object `T : Over S` corresponding to a morphism `p : X ⟶ S` are the type of morphisms `p^* M ⟶ p^* N`. We shall say that `F` satisfies the descent of morphisms for a Grothendieck topology `J` if these presheaves are all sheaves (typeclass `F.HasDescentOfMorphisms J`).
Co-authored-by: Christian Merten [christian@merten.dev](mailto:christian@merten.dev)
---
- [x] depends on: #24382
- [ ] depends on: #25971
[](https://gitpod.io/from-referrer/)
|
t-category-theory
merge-conflict
blocked-by-other-PR
WIP
|
474/0 |
Mathlib.lean,Mathlib/CategoryTheory/Bicategory/Functor/Cat.lean,Mathlib/CategoryTheory/Bicategory/Functor/Strict.lean,Mathlib/CategoryTheory/Sites/Descent/Morphisms.lean |
4 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
70-23480 2 months ago |
70-23481 2 months ago |
0-0 0 seconds |
26136 |
vasnesterov author:vasnesterov |
feat(Topology/Instances): Cantor set is homeomorphic to `ℕ → Bool` |
* Prove that `ofDigits` is a continuous map from `ℕ → Fin b` to `ℝ`.
* Prove that the Cantor set is homeomorphic to `ℕ → Bool`.
---
- [ ] depends on: #26096
[](https://gitpod.io/from-referrer/)
|
large-import
t-topology
merge-conflict
blocked-by-other-PR
|
614/0 |
Mathlib.lean,Mathlib/Algebra/Order/Floor/Semiring.lean,Mathlib/Data/Nat/Cast/Order/Field.lean,Mathlib/Data/Real/OfDigits.lean,Mathlib/Topology/Instances/CantorSet.lean,scripts/noshake.json |
6 |
8 |
['alreadydone', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'vasnesterov'] |
nobody |
70-20921 2 months ago |
70-20922 2 months ago |
0-128 2 minutes |
26149 |
vasnesterov author:vasnesterov |
feat(Topology): continuous surjection from Cantor set to Hilbert cube |
---
- [ ] depends on: #26136
[](https://gitpod.io/from-referrer/)
|
large-import
t-topology
merge-conflict
blocked-by-other-PR
|
752/0 |
Mathlib.lean,Mathlib/Algebra/Order/Floor/Semiring.lean,Mathlib/Data/Nat/Cast/Order/Field.lean,Mathlib/Data/Real/OfDigits.lean,Mathlib/Topology/Homeomorph/Defs.lean,Mathlib/Topology/Instances/CantorSet.lean,Mathlib/Topology/MetricSpace/HausdorffAlexandroff.lean,scripts/noshake.json |
8 |
5 |
['alreadydone', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'vasnesterov'] |
nobody |
70-20918 2 months ago |
70-20919 2 months ago |
0-2240 37 minutes |
26184 |
vasnesterov author:vasnesterov |
feat(Topology): every compact metric space is image of Cantor set |
---
- [ ] depends on: #26027
- [ ] depends on: #26149
[](https://gitpod.io/from-referrer/)
|
large-import
t-topology
merge-conflict
blocked-by-other-PR
|
869/0 |
Mathlib.lean,Mathlib/Algebra/Order/Floor/Semiring.lean,Mathlib/Data/Nat/Cast/Order/Field.lean,Mathlib/Data/Real/OfDigits.lean,Mathlib/Topology/Compactness/HilbertCubeEmbedding.lean,Mathlib/Topology/Homeomorph/Defs.lean,Mathlib/Topology/Instances/CantorSet.lean,Mathlib/Topology/MetricSpace/HausdorffAlexandroff.lean,scripts/noshake.json |
9 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
70-20913 2 months ago |
70-20914 2 months ago |
0-602 10 minutes |
26185 |
vasnesterov author:vasnesterov |
feat(Counterexamples): Peano curve |
Prove the existence of a continuous surjection from `unitInterval` onto `unitInterval × unitInterval`.
---
- [ ] depends on: #26184
[](https://gitpod.io/from-referrer/)
|
large-import
t-topology
merge-conflict
blocked-by-other-PR
|
927/0 |
Counterexamples.lean,Counterexamples/PeanoCurve.lean,Mathlib.lean,Mathlib/Algebra/Order/Floor/Semiring.lean,Mathlib/Data/Nat/Cast/Order/Field.lean,Mathlib/Data/Real/OfDigits.lean,Mathlib/Topology/Compactness/HilbertCubeEmbedding.lean,Mathlib/Topology/Homeomorph/Defs.lean,Mathlib/Topology/Instances/CantorSet.lean,Mathlib/Topology/MetricSpace/HausdorffAlexandroff.lean,scripts/noshake.json |
11 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
70-20912 2 months ago |
70-20913 2 months ago |
0-1381 23 minutes |
26395 |
winstonyin author:winstonyin |
feat: $C^1$ vector fields on compact manifolds define global flows |
This PR continues the work from #22254.
Original PR: https://github.com/leanprover-community/mathlib4/pull/22254
Any $C^1$ vector field on a compact boundaryless manifold `M` defines a unique global flow `ℝ → M → M`.
- [ ] depends on: #26394
---
[](https://gitpod.io/from-referrer/)
|
t-differential-geometry
merge-conflict
blocked-by-other-PR
WIP
|
841/406 |
Mathlib/Algebra/Order/Group/Abs.lean,Mathlib/Analysis/Normed/Group/Basic.lean,Mathlib/Analysis/ODE/PicardLindelof.lean,Mathlib/Geometry/Manifold/IntegralCurve/ExistUnique.lean,Mathlib/Order/Filter/Prod.lean,docs/1000.yaml,docs/undergrad.yaml |
7 |
4 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'winstonyin'] |
nobody |
70-20776 2 months ago |
70-20776 2 months ago |
0-52 52 seconds |
26465 |
joelriou author:joelriou |
feat(Algebra/Module): presentation of the `PiTensorProduct` |
Given a presentation of a finite number of `R`-modules `M i`, we obtain a presentation of the module `⨂[R] i, M i`.
---
- [ ] depends on: #26464
This PR continues the work from #18527.
Original PR: https://github.com/leanprover-community/mathlib4/pull/18527 |
file-removed
t-algebra
merge-conflict
blocked-by-other-PR
label:t-algebra$ |
525/4 |
Mathlib.lean,Mathlib/Algebra/Module/Presentation/PiTensor.lean,Mathlib/Analysis/NormedSpace/PiTensorProduct/ProjectiveSeminorm.lean,Mathlib/Data/Set/ComplSingletonLift.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 |
10 |
4 |
['github-actions', 'joelriou', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
70-20646 2 months ago |
70-20647 2 months ago |
0-2063 34 minutes |
26467 |
joelriou author:joelriou |
feat(LinearAlgebra): the tensor product of a finite family of free modules is free |
---
- [ ] depends on: #26464
- [ ] depends on: #26465
[](https://gitpod.io/from-referrer/)
|
file-removed
t-algebra
merge-conflict
blocked-by-other-PR
WIP
label:t-algebra$ |
607/7 |
Mathlib.lean,Mathlib/Algebra/Module/Presentation/Free.lean,Mathlib/Algebra/Module/Presentation/PiTensor.lean,Mathlib/Analysis/NormedSpace/PiTensorProduct/ProjectiveSeminorm.lean,Mathlib/Data/Set/ComplSingletonLift.lean,Mathlib/LinearAlgebra/PiTensorProduct/Basic.lean,Mathlib/LinearAlgebra/PiTensorProduct/Basis.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 |
12 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
70-20644 2 months ago |
70-20645 2 months ago |
0-2 2 seconds |
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
blocked-by-other-PR
|
467/0 |
Mathlib.lean,Mathlib/MeasureTheory/VectorMeasure/Variation/Defs.lean,Mathlib/MeasureTheory/VectorMeasure/Variation/Lemmas.lean |
3 |
1 |
['github-actions'] |
nobody |
70-4834 2 months ago |
70-5390 2 months ago |
15-66224 15 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
blocked-by-other-PR
|
680/0 |
Mathlib.lean,Mathlib/MeasureTheory/VectorMeasure/Variation/Defs.lean,Mathlib/MeasureTheory/VectorMeasure/Variation/Equiv.lean,Mathlib/MeasureTheory/VectorMeasure/Variation/Lemmas.lean |
4 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
70-4834 2 months ago |
70-5363 2 months ago |
15-65390 15 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
blocked-by-other-PR
|
432/0 |
Mathlib.lean,Mathlib/MeasureTheory/VectorMeasure/Variation/Defs.lean,Mathlib/MeasureTheory/VectorMeasure/Variation/Lemmas.lean |
3 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
70-4833 2 months ago |
70-5442 2 months ago |
15-68781 15 days |
24912 |
YaelDillies author:YaelDillies |
feat: affine monoids |
Define affine monoids as finitely generated cancellative torsion-free commutative monoids and prove a few of their basic properties:
* An affine monoid with no non-trivial unit is generated by its irreducible elements
* An affine monoid embeds into `ℤⁿ` for some `n`
* Let `M` be an affine monoid. If `R` is a domain, then so is `R[M]`.
From Toric
Co-authored-by: Patrick Luo
---
- [x] depends on: #24913
- [x] depends on: #24914
- [ ] depends on: #26110
[](https://gitpod.io/from-referrer/)
|
toric
t-algebra
blocked-by-other-PR
label:t-algebra$ |
214/0 |
Mathlib.lean,Mathlib/Algebra/AffineMonoid/Basic.lean,Mathlib/Algebra/AffineMonoid/Embedding.lean,Mathlib/Algebra/AffineMonoid/Irreducible.lean,Mathlib/Algebra/AffineMonoid/UniqueSums.lean |
5 |
15 |
['YaelDillies', 'b-mehta', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'smorel394'] |
nobody |
69-83730 2 months ago |
86-65942 2 months ago |
7-26907 7 days |
24627 |
pechersky author:pechersky |
feat(Topology/Algebra/Valued): `IsLinearTopology 𝒪[K] K` and `𝒪[K] 𝒪[K]` |
as well as
`IsLinearTopology ℤ_[p] ℤ_[p]`
---
[](https://gitpod.io/from-referrer/)
- [ ] depends on: #26829
|
t-topology
merge-conflict
awaiting-author
blocked-by-other-PR
|
376/30 |
Mathlib.lean,Mathlib/NumberTheory/Padics/LinearTopology.lean,Mathlib/RingTheory/Valuation/Basic.lean,Mathlib/RingTheory/Valuation/Integers.lean,Mathlib/Topology/Algebra/Valued/LinearTopology.lean,Mathlib/Topology/Algebra/Valued/LocallyCompact.lean,Mathlib/Topology/Algebra/Valued/ValuationTopology.lean,Mathlib/Topology/Algebra/Valued/ValuedField.lean |
8 |
41 |
['ADedecker', 'faenuccio', 'github-actions', 'leanprover-community-bot-assistant', 'loefflerd', 'mathlib4-dependent-issues-bot', 'pechersky'] |
nobody |
68-46482 2 months ago |
70-23475 2 months ago |
19-50489 19 days |
10654 |
smorel394 author:smorel394 |
feat(LinearAlgebra/{ExteriorPower,LinearIndependent,TensorPower}): define the exterior powers of a module and prove some of their basic properties |
This introduces the exterior powers of a module and proves some of their basic properties, in `LinearAlgebra/ExteriorPower/Basic.lean` and `LinearAlgebra/ExteriorPower/Generators.lean`. It also adds a lemma in `LinearAlgebra/LinearIndependent.lean` (`linearIndependent_of_dualFamily` : if a family of vectors admits a "dual" family of linear forms, then it is linearly independent) and a construction in `LinearAlgebra/TensorPower.lean` (`linearFormOfFamily` : the linear form on the tensor power of `M` obtained by multiplying a family of linear forms on `M`).
# Main definitions
## In `LinearAlgebra/ExteriorPower/Basic.lean`:
* `ExteriorPower R n M` is the `n`th exterior power of a `R`-module `M`, defined as `LinearMap.range (ExteriorAlgebra.ι R : M →ₗ[R] ExteriorAlgebra R M) ^ n`. We also introduce the notation `Λ[R]^n M` for `ExteriorPower R n M`.
* `ExteriorPower.ιMulti` is the canonical alternating map on `M` with values in `Λ[R]^n M`.
* `ExteriorPower.map`: functoriality of exterior powers with respect to linear maps between modules.
* `ExteriorPower.toTensorPower`: linear map from the `n`th exterior power to the `n`th
tensor power (coming from `MultilinearMap.alternatization` via the universal property of
exterior powers).
## In `LinearAlgebra/ExteriorPower/Generators.lean`:
* `ExteriorPower.BasisOfBasis`: If `b` is a basis of `M` (indexed by a linearly ordered type),
the basis of the `n`th exterior power of `M` formed by the `n`-fold exterior products of elements
of `b`.
# Main theorems
## In `LinearAlgebra/ExteriorPower/Basic.lean`:
* The image of `ExteriorPower.ιMulti` spans `Λ[R]^n M`.
* `ExteriorPower.liftAlternatingEquiv` (universal property of the `n`th exterior power of `M`):
the linear equivalence between linear maps from `Λ[R]^n M` to a module `N` and `n`-fold
alternating maps from `M` to `N`.
* `ExteriorPower.map_injective_field`: If `f : M →ₗ[R] N` is injective and `R` is a field, then
`ExteriorPower.map n f` is injective.
* `ExteriorPower.map_surjective`: If `f : M →ₗ[R] N` is surjective, then `ExteriorPower.map n f`
is surjective.
* `ExteriorPower.mem_exteriorPower_is_mem_finite`: Every element of `Λ[R]^n M` is in the image of
`Λ[R]^n P` for some finitely generated submodule `P` of `M`.
## In `LinearAlgebra/ExteriorPower/Generators.lean`:
* `ExteriorPower.Finite`: The `n`th exterior power of a finite module is a finite module.
* `ExteriorPower.span_top_of_span_top` and `ExteriorPower.span_top_of_span_top'`: If a family of
vectors spans `M`, then the family of its `n`-fold exterior products spans `Λ[R]^n M`. (We give
versions in the exterior algebra and in the exterior power.)
* `ExteriorPower.FreeOfFree`: If `M` is a free module, then so is its `n`th exterior power.
* `ExteriorPower.FinrankOfFiniteFree`: If `R` satisfies the strong rank condition and `M` is
finite free of rank `r`, then the `n`th exterior power of `M` is of finrank `Nat.choose r n`.
* `ExteriorPower.ιMulti_family_linearIndependent_field`: If `R` is a field, and if `v` is a
linearly independent family of vectors (indexed by a linearly ordered type), then the family of
its `n`-fold exterior products is also linearly independent.
- [x] depends on: #10744
- [ ] depends on: #11156
- [x] depends on: #18590
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebra
merge-conflict
please-adopt
blocked-by-other-PR
label:t-algebra$ |
739/0 |
Mathlib.lean,Mathlib/LinearAlgebra/ExteriorPower/Basic.lean,Mathlib/LinearAlgebra/ExteriorPower/Generators.lean,Mathlib/LinearAlgebra/LinearIndependent.lean,Mathlib/LinearAlgebra/TensorPower.lean |
5 |
46 |
['Ruben-VandeVelde', 'YaelDillies', 'bustercopley', 'eric-wieser', 'github-actions', 'joelriou', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'mattrobball', 'pink10000', 'smorel394'] |
eric-wieser assignee:eric-wieser |
60-19341 1 month ago |
282-51123 9 months ago |
22-67320 22 days |
26884 |
alreadydone author:alreadydone |
Universal cover |
---
- [ ] depends on: #24983
- [ ] depends on: #22771
- [ ] depends on: #22782
[](https://gitpod.io/from-referrer/)
|
t-topology
merge-conflict
blocked-by-other-PR
WIP
|
1126/359 |
Mathlib.lean,Mathlib/AlgebraicGeometry/ProjectiveSpectrum/StructureSheaf.lean,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/Data/Set/Operations.lean,Mathlib/Geometry/Manifold/Sheaf/Smooth.lean,Mathlib/Logic/Equiv/Basic.lean,Mathlib/Topology/Covering.lean,Mathlib/Topology/EtaleSpace.lean,Mathlib/Topology/FiberBundle/Trivialization.lean,Mathlib/Topology/Homotopy/HomotopyGroup.lean,Mathlib/Topology/Homotopy/Lifting.lean,Mathlib/Topology/Homotopy/Product.lean,Mathlib/Topology/IsLocalHomeomorph.lean,Mathlib/Topology/Sheaves/LocalPredicate.lean,Mathlib/Topology/Sheaves/Sheafify.lean,Mathlib/Topology/Sheaves/Stalks.lean |
20 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
60-4738 1 month ago |
65-64588 2 months ago |
0-0 0 seconds |
26950 |
alreadydone author:alreadydone |
Primitives of holomorphic functions and path integral |
---
- [ ] depends on: #22782
- [x] depends on: #24983
- [ ] depends on: #22771
[](https://gitpod.io/from-referrer/)
|
t-analysis
t-topology
merge-conflict
blocked-by-other-PR
WIP
|
1288/361 |
Mathlib.lean,Mathlib/AlgebraicGeometry/ProjectiveSpectrum/StructureSheaf.lean,Mathlib/AlgebraicTopology/FundamentalGroupoid/Basic.lean,Mathlib/AlgebraicTopology/FundamentalGroupoid/FundamentalGroup.lean,Mathlib/AlgebraicTopology/FundamentalGroupoid/InducedMaps.lean,Mathlib/AlgebraicTopology/FundamentalGroupoid/SimplyConnected.lean,Mathlib/Analysis/Complex/Primitive.lean,Mathlib/CategoryTheory/Groupoid.lean,Mathlib/Data/Set/Operations.lean,Mathlib/Geometry/Manifold/Sheaf/Smooth.lean,Mathlib/Logic/Equiv/Basic.lean,Mathlib/Topology/Covering.lean,Mathlib/Topology/EtaleSpace.lean,Mathlib/Topology/FiberBundle/Trivialization.lean,Mathlib/Topology/Homotopy/HomotopyGroup.lean,Mathlib/Topology/Homotopy/Lifting.lean,Mathlib/Topology/Homotopy/Product.lean,Mathlib/Topology/IsLocalHomeomorph.lean,Mathlib/Topology/Sheaves/LocalPredicate.lean,Mathlib/Topology/Sheaves/Sheafify.lean,Mathlib/Topology/Sheaves/Stalks.lean |
21 |
n/a |
['mathlib4-dependent-issues-bot'] |
nobody |
60-1179 1 month ago |
unknown |
unknown |
27070 |
vasnesterov author:vasnesterov |
golf: use `order` |
---
- [ ] depends on: #26580
[](https://gitpod.io/from-referrer/)
|
large-import
merge-conflict
blocked-by-other-PR
WIP
|
619/466 |
Mathlib.lean,Mathlib/Algebra/BigOperators/Intervals.lean,Mathlib/Algebra/ContinuedFractions/Computation/CorrectnessTerminating.lean,Mathlib/Algebra/ContinuedFractions/Computation/Translations.lean,Mathlib/Algebra/GeomSum.lean,Mathlib/Algebra/Group/Subgroup/Ker.lean,Mathlib/Algebra/Homology/ShortComplex/Ab.lean,Mathlib/Algebra/Lie/Ideal.lean,Mathlib/Algebra/Lie/IdealOperations.lean,Mathlib/Algebra/Lie/Semisimple/Basic.lean,Mathlib/Algebra/Lie/Subalgebra.lean,Mathlib/Algebra/Lie/Submodule.lean,Mathlib/Algebra/MvPolynomial/Degrees.lean,Mathlib/Algebra/MvPolynomial/Division.lean,Mathlib/Algebra/Order/Archimedean/Basic.lean,Mathlib/Algebra/Order/Group/Abs.lean,Mathlib/Algebra/Order/Group/Indicator.lean,Mathlib/Algebra/Order/Rearrangement.lean,Mathlib/Algebra/Order/Ring/IsNonarchimedean.lean,Mathlib/Algebra/Order/Star/Prod.lean,Mathlib/Algebra/Order/ToIntervalMod.lean,Mathlib/Algebra/Polynomial/CoeffMem.lean,Mathlib/Algebra/Polynomial/Degree/Definitions.lean,Mathlib/Algebra/Polynomial/Inductions.lean,Mathlib/Algebra/Polynomial/Monic.lean,Mathlib/Algebra/Polynomial/Sequence.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Affine/Point.lean,Mathlib/AlgebraicGeometry/ValuativeCriterion.lean,Mathlib/AlgebraicTopology/SimplicialObject/Split.lean,Mathlib/Analysis/Calculus/Deriv/MeanValue.lean,Mathlib/Analysis/Calculus/UniformLimitsDeriv.lean,Mathlib/Analysis/ConstantSpeed.lean,Mathlib/Analysis/Convex/StrictConvexBetween.lean,Mathlib/Analysis/Convex/Uniform.lean,Mathlib/Analysis/Convolution.lean,Mathlib/Analysis/Distribution/SchwartzSpace.lean,Mathlib/Analysis/InnerProductSpace/Orthogonal.lean,Mathlib/Analysis/InnerProductSpace/Projection.lean,Mathlib/Analysis/Matrix.lean,Mathlib/Analysis/MeanInequalities.lean,Mathlib/Analysis/MeanInequalitiesPow.lean,Mathlib/Analysis/Meromorphic/FactorizedRational.lean,Mathlib/Analysis/Meromorphic/NormalForm.lean,Mathlib/Analysis/Normed/Group/Seminorm.lean,Mathlib/Analysis/SpecialFunctions/Complex/Arg.lean,Mathlib/Analysis/SpecialFunctions/Log/Base.lean,Mathlib/Analysis/SpecialFunctions/PolarCoord.lean,Mathlib/CategoryTheory/SmallObject/Iteration/ExtendToSucc.lean,Mathlib/CategoryTheory/Subpresheaf/Equalizer.lean,Mathlib/Combinatorics/Additive/Corner/Roth.lean,Mathlib/Combinatorics/SimpleGraph/Clique.lean,Mathlib/Combinatorics/SimpleGraph/Coloring.lean,Mathlib/Combinatorics/SimpleGraph/Connectivity/Connected.lean,Mathlib/Combinatorics/SimpleGraph/Girth.lean,Mathlib/Computability/AkraBazzi/AkraBazzi.lean,Mathlib/Computability/AkraBazzi/GrowsPolynomially.lean,Mathlib/Computability/Partrec.lean,Mathlib/Data/ENNReal/Inv.lean,Mathlib/Data/EReal/Operations.lean,Mathlib/Data/FinEnum/Option.lean,Mathlib/Data/Finset/Lattice/Fold.lean,Mathlib/Data/Fintype/Perm.lean,Mathlib/Data/Int/WithZero.lean,Mathlib/Data/List/MinMax.lean,Mathlib/Data/Matroid/Basic.lean,Mathlib/Data/Nat/Choose/Central.lean,Mathlib/Data/Nat/Digits/Defs.lean,Mathlib/Data/Nat/Factors.lean,Mathlib/Data/Nat/Multiplicity.lean,Mathlib/Data/Nat/PartENat.lean,Mathlib/Data/PNat/Basic.lean,Mathlib/Data/Rat/Floor.lean,Mathlib/Data/Set/MemPartition.lean,Mathlib/Data/Sign.lean,Mathlib/Dynamics/TopologicalEntropy/Subset.lean,Mathlib/FieldTheory/Relrank.lean,Mathlib/Geometry/Manifold/Instances/Real.lean,Mathlib/Geometry/Manifold/IsManifold/Basic.lean,Mathlib/Geometry/RingedSpace/Basic.lean,Mathlib/GroupTheory/Perm/Sign.lean,Mathlib/LinearAlgebra/AffineSpace/AffineSubspace/Defs.lean,Mathlib/LinearAlgebra/AffineSpace/FiniteDimensional.lean,Mathlib/LinearAlgebra/ExteriorPower/Pairing.lean,Mathlib/LinearAlgebra/Matrix/Block.lean,Mathlib/LinearAlgebra/QuadraticForm/Basic.lean,Mathlib/MeasureTheory/Constructions/BorelSpace/Real.lean,Mathlib/MeasureTheory/Covering/Besicovitch.lean,Mathlib/MeasureTheory/Covering/Differentiation.lean,Mathlib/MeasureTheory/Covering/LiminfLimsup.lean,Mathlib/MeasureTheory/Covering/Vitali.lean,Mathlib/MeasureTheory/Function/AEEqFun.lean,Mathlib/MeasureTheory/Function/AEEqOfIntegral.lean,Mathlib/MeasureTheory/Function/AEEqOfLIntegral.lean,Mathlib/MeasureTheory/Function/ConvergenceInMeasure.lean,Mathlib/MeasureTheory/Function/Jacobian.lean,Mathlib/MeasureTheory/Function/LpSeminorm/Basic.lean,Mathlib/MeasureTheory/Function/LpSeminorm/CompareExp.lean,Mathlib/MeasureTheory/Function/SimpleFunc.lean,Mathlib/MeasureTheory/Function/UniformIntegrable.lean,Mathlib/MeasureTheory/Integral/Bochner/VitaliCaratheodory.lean |
224 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
59-70992 1 month ago |
59-70993 1 month ago |
0-10 10 seconds |
26886 |
pechersky author:pechersky |
feat(NumberTheory/Padics/ValuativeRel): ValuativeRel ℚ_[p] |
as well as instances for IsRankLeOne, IsNontrivial, IsDiscrete
---
[](https://gitpod.io/from-referrer/)
- [ ] depends on: #26827 |
t-algebra
t-analysis
t-number-theory
merge-conflict
blocked-by-other-PR
WIP
label:t-algebra$ |
310/25 |
Mathlib.lean,Mathlib/Analysis/Normed/ValuativeRel.lean,Mathlib/NumberTheory/Padics/ValuativeRel.lean,Mathlib/Topology/Algebra/Valued/ValuativeRel.lean |
4 |
4 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
59-42609 1 month ago |
59-42609 1 month ago |
0-1386 23 minutes |
26983 |
mans0954 author:mans0954 |
feat(Order/LatticeElements): distributive, standard and neutral elements of a lattice |
Defines distributive, standard and neutral elements of a lattice and gives equivalent conditions.
---
- [ ] depends on: #26836
[](https://gitpod.io/from-referrer/)
|
t-order
blocked-by-other-PR
|
287/0 |
Mathlib.lean,Mathlib/Order/Lattice.lean,Mathlib/Order/LatticeElements.lean,docs/references.bib |
4 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
58-12569 1 month ago |
58-17210 1 month ago |
0-9 9 seconds |
25834 |
Rida-Hamadani author:Rida-Hamadani |
feat(SimpleGraph): girth-diameter inequality |
This is a useful inequality that comes up in proofs related to Moore graphs, cages, SRGs, and so on.
---
- [x] depends on: #26380
- [x] depends on: #25650
- [ ] depends on: #26614
[](https://gitpod.io/from-referrer/)
|
t-combinatorics
blocked-by-other-PR
WIP
|
825/0 |
Mathlib.lean,Mathlib/Combinatorics/SimpleGraph/GirthDiam.lean |
2 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
57-559 1 month ago |
80-40353 2 months ago |
0-28 28 seconds |
26973 |
peabrainiac author:peabrainiac |
feat(Geometry/Diffeology): diffeologies generated from sets of plots |
Introduces diffeologies generated from sets of plots, shows that this defines a Galois insertion, and concludes that the diffeologies on a type form a complete lattice.
---
This PR continues the work from #22724.
- [ ] depends on: #26484 |
t-differential-geometry
blocked-by-other-PR
|
629/0 |
Mathlib.lean,Mathlib/Geometry/Diffeology/Basic.lean,docs/references.bib |
3 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'peabrainiac'] |
nobody |
56-48575 1 month ago |
64-64249 2 months ago |
0-785 13 minutes |
27258 |
JovanGerb author:JovanGerb |
Imo2020 q6 |
Original PR: #23431
This PR adds a solution to IMO 2020 Q6. It follows the solution that I found when I was participating in the IMO. I used the statement formalization that was given by @jsm28.
The function `project a b p` that is defined here is the same as `signedDist a p (b -ᵥ a)` defined in #27260.
---
- [ ] depends on: #27257
[](https://gitpod.io/from-referrer/)
|
IMO
blocked-by-other-PR
|
367/0 |
Archive.lean,Archive/Imo/Imo2020Q6.lean |
2 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
56-40277 1 month ago |
56-63494 1 month ago |
0-1307 21 minutes |
27274 |
peabrainiac author:peabrainiac |
feat(Geometry/Diffeology): continuous diffeologies & D-topology-lemmas |
Introduces the continuous diffeology on topological spaces and the Galois connection between it and the D-topology, and then uses it to prove a few more lemmas about the D-topology.
---
Aside from being useful for defining a right adjoint of the D-topology functor later, this is a prerequisite for correctly defining coinduced diffeologies (namely in such a way that the D-topology is defeq to the coinduced topology) and thus also for most constructions of diffeological spaces.
- [ ] depends on: #26973
[](https://gitpod.io/from-referrer/)
|
t-differential-geometry
blocked-by-other-PR
|
766/0 |
Mathlib.lean,Mathlib/Geometry/Diffeology/Basic.lean,Mathlib/Geometry/Diffeology/Continuous.lean,docs/references.bib |
4 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
56-29268 1 month ago |
56-29269 1 month ago |
0-1796 29 minutes |
25848 |
joelriou author:joelriou |
feat/refactor: redefinition of homology + derived categories |
This PR contains a redefinition of homology, theorems about localization of categories, including triangulated categories, a construction of the derived category of an abelian category, derived functors, spectral sequences, etc. (This is made a PR only to facilitate navigation in the code of this branch.)
This formalization is outlined in the paper _Formalization of derived categories in Lean/mathlib_ https://hal.science/hal-04546712
The homology of `ShortComplex C` (diagrams of two composable morphisms whose composition is zero) is developed in `Algebra.Homology.ShortComplex`. The files in that folder have been added one by one in separate PRs, and then, the current definition of `homology` has been replaced by this new definition in a refactor PR.
Homology refactor:
* #4203
* #4204
* #4388
* #4609
* #4645
* #4787
* #4853
* #5250
* #5674
* #6008
* #6039
* #6089
* #6227
* #6230
* #6231
* #6245
* #6267
* #6279
* #6324
* #6443
* #6586
* #6994
* #7042
* #7047
* #7052
* #7192
* #7193
* #7194
* #7195
* #7197
* #7256
* #7262
* #7280
* #7623
* #7624
* #7806
* #7816
* #7817
* #7821
* #7954
* #7966
* #7993
* #7995
* #7996
* #7997
* #8058
* #8060
* #8069
* #8079
* #8081
* #8084
* #8091
* #8113
* #8114
* #8152
* #8159
* #8174
* #8200
* #8206
* #8208
* #8472
* #8468
* #8475
* #8490
* #8491
* #8507
* #8512
* #8593
* #8595
* #8706
* #8765
* #8766
* #8845
* #9022
* #12649
* #12638
Homological complexes:
* #9333
* #9335
* #9331
Localization of categories:
* #6233
* #6235
* #6236
* #6867
* #6869
* #6887
* #6882
* #8041
* #8055
* #8069
* #8516
* #8864
* #8865
* #9702
* #9692
* #10606
* #10607
* #11721
* #11728
* #11737
* #12728
Shifts on categories:
* #4429
* #6652
* #6653
* #6655
* #7268
* #7270
* #9001
* #11764
Triangulated categories:
* #6377
* #6688
* #6815
* #7053
* #7324
* #7327
* #7336
* #7626
* #7641
* #9049
* #9073
* #10527
* #11738
* #11740
* #11759
* #11786
* #11789
* #11805
* #12619
Construction of the derived category:
* #6626
* #6701
* #6720
* #6894
* #7048
* #7049
* #7050
* #7201
* #7656
* #8937
* #8966
* #8969
* #8970
* #9054
* #9447
* #8951
* #9483
* #9508
* #9509
* #9592
* #9614
* #9615
* #9032
* #9370
* #9550
* #9686
* #9660
* #11760
* #11782
* #11806
Derived functors:
* #10195
* #10270
* #10301
* #10384
* #10413
* #12168
* #12627
* #12631
* #12633
* #12785
* #12788
Refactor of Ext-groups:
* #12607
- [ ] depends on: #24309
- [ ] depends on: #24275
- [x] depends on: #24191
- [ ] depends on: #23797
- [x] depends on: #22586
- [ ] depends on: #22556
- [ ] depends on: #22547
- [ ] depends on: #22539
- [ ] depends on: #22508
- [ ] depends on: #22450
- [ ] depends on: #23915
---
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #4197.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/4197* |
large-import
t-topology
t-category-theory
merge-conflict
blocked-by-other-PR
WIP
|
41795/490 |
Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Free.lean,Mathlib/Algebra/Category/ModuleCat/LeftResolutions.lean,Mathlib/Algebra/Homology/Additive.lean,Mathlib/Algebra/Homology/BicomplexColumns.lean,Mathlib/Algebra/Homology/BicomplexRows.lean,Mathlib/Algebra/Homology/Bifunctor.lean,Mathlib/Algebra/Homology/BifunctorColimits.lean,Mathlib/Algebra/Homology/BifunctorCommShift.lean,Mathlib/Algebra/Homology/BifunctorFlip.lean,Mathlib/Algebra/Homology/BifunctorHomotopy.lean,Mathlib/Algebra/Homology/BifunctorMappingCone.lean,Mathlib/Algebra/Homology/BifunctorShift.lean,Mathlib/Algebra/Homology/BifunctorSingle.lean,Mathlib/Algebra/Homology/BifunctorTriangulated.lean,Mathlib/Algebra/Homology/CategoryWithHomology.lean,Mathlib/Algebra/Homology/CochainComplexMinus.lean,Mathlib/Algebra/Homology/ComplexShape.lean,Mathlib/Algebra/Homology/ComplexShapeSigns.lean,Mathlib/Algebra/Homology/ConnectShortExact.lean,Mathlib/Algebra/Homology/DerivedCategory/Basic.lean,Mathlib/Algebra/Homology/DerivedCategory/DerivabilityStructureInjectives.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/Linear.lean,Mathlib/Algebra/Homology/DerivedCategory/Fractions.lean,Mathlib/Algebra/Homology/DerivedCategory/FullyFaithful.lean,Mathlib/Algebra/Homology/DerivedCategory/HomologySequence.lean,Mathlib/Algebra/Homology/DerivedCategory/Linear.lean,Mathlib/Algebra/Homology/DerivedCategory/Minus.lean,Mathlib/Algebra/Homology/DerivedCategory/Monoidal.lean,Mathlib/Algebra/Homology/DerivedCategory/Plus.lean,Mathlib/Algebra/Homology/DerivedCategory/RightDerivedFunctorPlus.lean,Mathlib/Algebra/Homology/DerivedCategory/SingleTriangle.lean,Mathlib/Algebra/Homology/DerivedCategory/SpectralObject.lean,Mathlib/Algebra/Homology/DerivedCategory/TStructure.lean,Mathlib/Algebra/Homology/Double.lean,Mathlib/Algebra/Homology/DoubleHomology.lean,Mathlib/Algebra/Homology/Embedding/CochainComplex.lean,Mathlib/Algebra/Homology/Embedding/CochainComplexTrunc.lean,Mathlib/Algebra/Homology/Embedding/ComplementaryTrunc.lean,Mathlib/Algebra/Homology/Embedding/ExtendMap.lean,Mathlib/Algebra/Homology/Embedding/HomEquiv.lean,Mathlib/Algebra/Homology/Embedding/RestrictionHomology.lean,Mathlib/Algebra/Homology/Embedding/StupidFiltration.lean,Mathlib/Algebra/Homology/Embedding/StupidTrunc.lean,Mathlib/Algebra/Homology/Embedding/TruncGE.lean,Mathlib/Algebra/Homology/Embedding/TruncLE.lean,Mathlib/Algebra/Homology/Embedding/TruncLEHomology.lean,Mathlib/Algebra/Homology/ExactSequence.lean,Mathlib/Algebra/Homology/ExactSequenceFour.lean,Mathlib/Algebra/Homology/Factorizations/Basic.lean,Mathlib/Algebra/Homology/Factorizations/CM5a.lean,Mathlib/Algebra/Homology/Factorizations/CM5b.lean,Mathlib/Algebra/Homology/HomologicalBicomplex.lean,Mathlib/Algebra/Homology/HomologicalComplex.lean,Mathlib/Algebra/Homology/HomologicalComplexFunctorEquiv.lean,Mathlib/Algebra/Homology/HomologicalComplexLimits.lean,Mathlib/Algebra/Homology/HomologicalComplexLimitsEventuallyConstant.lean,Mathlib/Algebra/Homology/Homology.lean,Mathlib/Algebra/Homology/HomologySequence.lean,Mathlib/Algebra/Homology/HomologySequenceLemmas.lean,Mathlib/Algebra/Homology/Homotopy.lean,Mathlib/Algebra/Homology/HomotopyCategory.lean,Mathlib/Algebra/Homology/HomotopyCategory/Cylinder.lean,Mathlib/Algebra/Homology/HomotopyCategory/DegreewiseSplit.lean,Mathlib/Algebra/Homology/HomotopyCategory/Devissage.lean,Mathlib/Algebra/Homology/HomotopyCategory/HomComplex.lean,Mathlib/Algebra/Homology/HomotopyCategory/HomComplexShift.lean,Mathlib/Algebra/Homology/HomotopyCategory/KInjective.lean,Mathlib/Algebra/Homology/HomotopyCategory/MappingCone.lean,Mathlib/Algebra/Homology/HomotopyCategory/Minus.lean,Mathlib/Algebra/Homology/HomotopyCategory/Monoidal.lean,Mathlib/Algebra/Homology/HomotopyCategory/MonoidalTriangulated.lean,Mathlib/Algebra/Homology/HomotopyCategory/Plus.lean,Mathlib/Algebra/Homology/HomotopyCategory/PreservesQuasiIso.lean,Mathlib/Algebra/Homology/HomotopyCategory/Pretriangulated.lean,Mathlib/Algebra/Homology/HomotopyCategory/Shift.lean,Mathlib/Algebra/Homology/HomotopyCategory/ShiftSequence.lean,Mathlib/Algebra/Homology/HomotopyCategory/ShortExact.lean,Mathlib/Algebra/Homology/HomotopyCategory/SingleFunctors.lean,Mathlib/Algebra/Homology/HomotopyCategory/SpectralObject.lean,Mathlib/Algebra/Homology/HomotopyFiber.lean,Mathlib/Algebra/Homology/LeftResolutions/Basic.lean,Mathlib/Algebra/Homology/LeftResolutions/CochainComplex.lean,Mathlib/Algebra/Homology/LeftResolutions/CochainComplexMinus.lean,Mathlib/Algebra/Homology/LeftResolutions/Reduced.lean,Mathlib/Algebra/Homology/LeftResolutions/Transport.lean,Mathlib/Algebra/Homology/Localization.lean,Mathlib/Algebra/Homology/Monoidal.lean,Mathlib/Algebra/Homology/ObjectProperty.lean,Mathlib/Algebra/Homology/PreservesQuasiIso.lean,Mathlib/Algebra/Homology/QuasiIso.lean,Mathlib/Algebra/Homology/Refinements.lean,Mathlib/Algebra/Homology/ShortComplex/Abelian.lean,Mathlib/Algebra/Homology/ShortComplex/Basic.lean,Mathlib/Algebra/Homology/ShortComplex/Exact.lean,Mathlib/Algebra/Homology/ShortComplex/FiveLemma.lean,Mathlib/Algebra/Homology/ShortComplex/FourLemma.lean,Mathlib/Algebra/Homology/ShortComplex/HomologicalComplex.lean,Mathlib/Algebra/Homology/ShortComplex/Images.lean,Mathlib/Algebra/Homology/ShortComplex/Preadditive.lean |
295 |
n/a |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
51-70620 1 month ago |
unknown |
unknown |
27416 |
joelriou author:joelriou |
feat(Algebra/Homology): Ext modules |
In this PR, we show that if `C` is a `R`-linear abelian category, then there is a `R`-module structure on the groups `Ext X Y n` for `X` and `Y` in `C` and `n : ℕ`.
---
- [ ] depends on: #26031
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-category-theory
blocked-by-other-PR
WIP
label:t-algebra$ |
172/0 |
Mathlib.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/Linear.lean,Mathlib/Algebra/Homology/DerivedCategory/Linear.lean,Mathlib/Algebra/Homology/HomotopyCategory/Shift.lean,Mathlib/Algebra/Homology/HomotopyCategory/SingleFunctors.lean |
5 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
51-17529 1 month ago |
51-17529 1 month ago |
0-146 2 minutes |
19607 |
madvorak author:madvorak |
Block matrix totally unimodular |
---
Discussion: https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/TU.20block.20matrix.20.2319607
- [ ] depends on: #19323
- [ ] depends on: #20428
- [ ] depends on: #20433
[](https://gitpod.io/from-referrer/)
|
merge-conflict
blocked-by-other-PR
WIP
|
156/0 |
Mathlib.lean,Mathlib/Data/Sum/Decompose.lean,Mathlib/LinearAlgebra/Matrix/Determinant/TotallyUnimodular.lean |
3 |
11 |
['github-actions', 'jcommelin', 'leanprover-community-bot-assistant', 'madvorak', 'mathlib4-dependent-issues-bot'] |
nobody |
51-3550 1 month ago |
51-3551 1 month ago |
0-0 0 seconds |
26987 |
joelriou author:joelriou |
chore: deprecating module LinearAlgebra.PiTensorProduct |
---
- [ ] depends on: #26464
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
blocked-by-other-PR
WIP
label:t-algebra$ |
1209/934 |
Mathlib.lean,Mathlib/Analysis/NormedSpace/PiTensorProduct/ProjectiveSeminorm.lean,Mathlib/Data/SubtypeNeLift.lean,Mathlib/LinearAlgebra/PiTensorProduct.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 |
10 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
51-1950 1 month ago |
51-1950 1 month ago |
0-2 2 seconds |
24668 |
robertmaxton42 author:robertmaxton42 |
feat(LinearAlgebra): add inductive principle for the free product of algebras |
* Add `FreeProduct.inductionOn` and `.asPowers.inductionOn`.
- [ ] depends on: #24532
---
* `simp↓` on `empty_rel'_bot`: the LHS is indeed not in simp-normal form, but `simp` can't solve the full lemma (if only because `Function.onFun` isn't marked `@[simp]`) and the actual simp-normal form of `rel'` isn't terribly useful for humans. Since I do expect users to type `rel' R A` by hand, I claim this use of `simp↓` is justified.
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
blocked-by-other-PR
label:t-algebra$ |
205/9 |
Mathlib/LinearAlgebra/FreeProduct/Basic.lean |
1 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
49-31519 1 month ago |
49-31520 1 month ago |
0-333 5 minutes |
27025 |
grunweg author:grunweg |
feat: Gram-Schmidt procedure on smooth vector bundles yields smooth sections |
For the Gram-Schmidt process on a vector bundle, deduce that smoothness of the bundle metric implies smoothness of the resulting sections.
From the path towards geodesics and the Levi-Civita connection.
Co-authored-by: Patrick Massot
---
A few sorries remain to prove the continuous case.
- [ ] depends on: #27021
- [x] depends on: #27023
- [ ] depends on: #27024
[](https://gitpod.io/from-referrer/)
|
t-differential-geometry
blocked-by-other-PR
|
927/11 |
Mathlib.lean,Mathlib/Analysis/InnerProductSpace/GramSchmidtOrtho.lean,Mathlib/Geometry/Manifold/Elaborators.lean,Mathlib/Geometry/Manifold/Traces.lean,Mathlib/Geometry/Manifold/VectorBundle/GramSchmidtOrtho.lean,scripts/noshake.json |
6 |
5 |
['faenuccio', 'github-actions', 'grunweg', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
44-60672 1 month ago |
45-73500 1 month ago |
0-316 5 minutes |
27694 |
grunweg author:grunweg |
feat: Gram-Schmidt orthonormalisation preserves continuity of sections |
provided the bundle metric used in the process is continuous.
From the path towards geodesics and the Levi-Civita connection.
Co-authored-by: Patrick Massot [patrickmassot@free.fr](mailto:patrickmassot@free.fr)
---
- [ ] depends on: #27024
- [ ] depends on: #27021
Baby version of #27025.
[](https://gitpod.io/from-referrer/)
|
t-differential-geometry
blocked-by-other-PR
|
390/11 |
Mathlib.lean,Mathlib/Analysis/InnerProductSpace/GramSchmidtOrtho.lean,Mathlib/Geometry/Manifold/VectorBundle/GramSchmidtOrtho.lean,scripts/noshake.json |
4 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
44-59943 1 month ago |
44-59943 1 month ago |
0-696 11 minutes |
26264 |
EtienneC30 author:EtienneC30 |
feat: characteristic function on product space |
The characteristic function of a measure is a product of characteristic functions if and only if the measure is a product measure. We prove this for Hilbert spaces and Banach spaces equipped with any Lp norm.
---
- [x] depends on: #26248
- [x] depends on: #26249
- [ ] depends on: #26498
[](https://gitpod.io/from-referrer/)
|
t-measure-probability
merge-conflict
blocked-by-other-PR
|
279/12 |
Mathlib/Analysis/Normed/Lp/PiLp.lean,Mathlib/Analysis/Normed/Lp/ProdLp.lean,Mathlib/Analysis/Normed/Lp/WithLp.lean,Mathlib/LinearAlgebra/Pi.lean,Mathlib/MeasureTheory/Measure/CharacteristicFunction.lean,Mathlib/Topology/Algebra/Module/LinearMapPiProd.lean |
6 |
6 |
['EtienneC30', 'RemyDegenne', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib-bors', 'mathlib4-dependent-issues-bot'] |
nobody |
43-84461 1 month ago |
43-84462 1 month ago |
0-83071 23 hours |
26269 |
EtienneC30 author:EtienneC30 |
feat: links between characteristic function and independence |
Prove several results of the form: random variables are independent if and only if their joint characteristic function is equal to the product of the characteristic functions. More specifically, prove this in Hilbert spaces for two variables
and a finite family of variables. Same in Banach spaces, with an arbitrary Lp norm.
---
- [ ] depends on: #26264
[](https://gitpod.io/from-referrer/)
|
t-measure-probability
merge-conflict
blocked-by-other-PR
|
489/12 |
Mathlib.lean,Mathlib/Analysis/Normed/Lp/PiLp.lean,Mathlib/Analysis/Normed/Lp/ProdLp.lean,Mathlib/Analysis/Normed/Lp/WithLp.lean,Mathlib/LinearAlgebra/Pi.lean,Mathlib/MeasureTheory/Measure/CharacteristicFunction.lean,Mathlib/Probability/Independence/CharacteristicFunction.lean,Mathlib/Topology/Algebra/Module/LinearMapPiProd.lean |
8 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
43-84459 1 month ago |
43-84460 1 month ago |
3-13100 3 days |
10006 |
jstoobysmith author:jstoobysmith |
feat(AlgebraicTopology): homotopy in quasicategories |
Defined a homotopy between two 1-simplicies in a quasicategories, and proved the property of being homotopic forms an equivalence relation.
---
- [ ] depends on: #9935
[](https://gitpod.io/from-referrer/)
|
t-algebraic-topology
new-contributor
merge-conflict
awaiting-author
blocked-by-other-PR
|
898/1 |
Mathlib.lean,Mathlib/AlgebraicTopology/Homotopy.lean,Mathlib/AlgebraicTopology/SimplexCategory.lean,Mathlib/AlgebraicTopology/SimplicialSet.lean |
4 |
3 |
['joelriou', 'leanprover-community-mathlib4-bot'] |
nobody |
43-81425 1 month ago |
43-81425 1 month ago |
0-0 0 seconds |
25740 |
robin-carlier author:robin-carlier |
feat(AlgebraicTopology/SimplexCategory/GeneratorsRelations): `SimplexCategoryGenRel.toSimplexCategory` is an equivalence |
We use the normal forms for morphisms in `SimplexCategoryGenRel` to prove that `SimplexCategoryGenRel.toSimplexCategory` is an equivalence. We prove in order that there exists unique lifts in `SimplexCategoryGenRel` of mono (resp. epis) in `SimplexCategory`, and use this to deduce fully faithfulness of `SimplexCategoryGenRel.toSimplexCategory` thanks to the existing epi-mono factorisation in `SimplexCategory`.
Part of a series of PR formalising that `SimplexCategoryGenRel` is equivalent to `SimplexCategory`.
---
- [ ] depends on: #25737
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #21747.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/21747* |
t-algebraic-topology
large-import
blocked-by-other-PR
|
942/9 |
Mathlib.lean,Mathlib/AlgebraicTopology/SimplexCategory/GeneratorsRelations/Equivalence.lean,Mathlib/AlgebraicTopology/SimplexCategory/GeneratorsRelations/NormalForms.lean |
3 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
43-81384 1 month ago |
43-81385 1 month ago |
0-2 2 seconds |
26399 |
ChrisHughes24 author:ChrisHughes24 |
refactor(ModelTheory): tidy up proof of Ax-Grothendieck with definable functions |
I migrated this PR by hand instead of using the script.
---
- [x] depends on: #20166
- [x] depends on: #20161
- [x] depends on: #20115
- [x] depends on: #20174
- [x] depends on: #20175
- [x] depends on: #20180
- [x] depends on: #21948
- [ ] depends on: #26398
[](https://gitpod.io/from-referrer/)
|
t-logic
blocked-by-other-PR
|
639/60 |
Mathlib.lean,Mathlib/FieldTheory/AxGrothendieck.lean,Mathlib/ModelTheory/FunctionalFormula.lean |
3 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
42-75626 1 month ago |
42-75699 1 month ago |
0-2300 38 minutes |
20008 |
FLDutchmann author:FLDutchmann |
feat(NumberTheory): Selberg sieve |
This PR is a working draft of the full proof of the fundamental theorem of the Selberg sieve. I will create dependent PRs as I clean up the code.
This work was used in the first proof of the prime number theorem in PNT+.
---
- [x] depends on: #20025
- [x] depends on: #20026
- [x] depends on: #20779
- [x] depends on: #21880
- [ ] depends on: #27702
- [ ] depends on: #27707
[](https://gitpod.io/from-referrer/)
|
t-analysis
t-number-theory
merge-conflict
awaiting-author
blocked-by-other-PR
|
937/0 |
Mathlib/NumberTheory/SelbergSieve/Basic.lean,Mathlib/NumberTheory/SelbergSieve/Selberg.lean,docs/references.bib |
3 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
42-66932 1 month ago |
42-66933 1 month ago |
0-0 0 seconds |
27838 |
CBirkbeck author:CBirkbeck |
feat(NumberTheory/LSeries/RiemannZeta): add tsum over ints lemma. |
---
- [ ] depends on: #27841
[](https://gitpod.io/from-referrer/)
|
t-number-theory
blocked-by-other-PR
|
63/2 |
Mathlib/NumberTheory/LSeries/RiemannZeta.lean,Mathlib/Topology/Algebra/InfiniteSum/NatInt.lean |
2 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
42-64211 1 month ago |
42-64273 1 month ago |
0-1182 19 minutes |
27228 |
themathqueen author:themathqueen |
feat: defining the inner product on tensor products |
This defines the inner product on tensor product spaces. Also defines `OrthonormalBasis.tensorProduct`.
The implementation is based on [here](https://github.com/ocfnash/lean-shannon-lovasz/blob/e63e535599ffb3c2a7e995e1621847693dd68fab/src/to_mathlib/analysis/inner_product_space/tensor_product.lean#L404) (by @jjaassoonn), which defines the inner product on real tensor product spaces. The exact same implementation also applies for the general case.
Closes #6020
---
- [ ] depends on: #27353
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-analysis
blocked-by-other-PR
label:t-algebra$ |
376/10 |
Mathlib.lean,Mathlib/Analysis/InnerProductSpace/TensorProduct.lean,Mathlib/LinearAlgebra/FiniteDimensional/Basic.lean,Mathlib/LinearAlgebra/TensorProduct/Basic.lean,Mathlib/LinearAlgebra/TensorProduct/Basis.lean |
5 |
5 |
['eric-wieser', 'github-actions', 'mathlib4-dependent-issues-bot', 'themathqueen'] |
nobody |
40-2140 1 month ago |
40-2140 1 month ago |
0-1325 22 minutes |
25486 |
VTrelat author:VTrelat |
feat(SetTheory/ZFC/Integers): define integers in ZFC |
Extend the model of ZFC with integers following the converse direction as for naturals. We first define a type and then build a set. We finally show that both representations have coercions in both direction:
- define a proper type `ZFInt` representing integers based on `ZFNat × ZFNat` and following the usual construction of integers
- add theorems on usual algebraic properties of integers
- define a set `Int` and show that it matches-i.e. that it is isomorphic to-the type `ZFInt`
---
[](https://gitpod.io/from-referrer/)
- [ ] depends on: #25483
- [ ] depends on: #25485 |
t-set-theory
new-contributor
merge-conflict
blocked-by-other-PR
|
2003/0 |
Mathlib/Data/Set/Prod.lean,Mathlib/SetTheory/ZFC/Basic.lean,Mathlib/SetTheory/ZFC/Booleans.lean,Mathlib/SetTheory/ZFC/Integers.lean |
4 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
40-1589 1 month ago |
40-1589 1 month ago |
0-2067 34 minutes |
25484 |
VTrelat author:VTrelat |
feat(SetTheory/ZFC/Booleans): define Boolean algebra in ZFC |
Extend the model of ZFC with Boolean algebra:
- define a set 𝔹 of booleans
- define a proper type `ZFBool` representing booleans
- add theorems on usual algebraic properties of booleans
- provide usual boolean notations like `⊤`, `⊥`, `∧`, `∨`, etc.
---
[](https://gitpod.io/from-referrer/)
- [ ] depends on: #25483 |
t-set-theory
new-contributor
merge-conflict
blocked-by-other-PR
|
619/0 |
Mathlib/Data/Set/Prod.lean,Mathlib/SetTheory/ZFC/Basic.lean,Mathlib/SetTheory/ZFC/Booleans.lean |
3 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
40-1580 1 month ago |
40-1580 1 month ago |
0-1523 25 minutes |
25427 |
Paul-Lez author:Paul-Lez |
feat(Analysis/Calculus/PartialDerivatives): Propose notation for partial derivatives. |
This PR introduces a notation for partial derivatives, taken with respect to a canonical basis. The idea here is that this might be useful for e.g. writing down PDEs. The notation allows use to write things like
```lean
-- The canonical basis for `ℝ × ℝ` is indexed by `Fin 0` so `∂₀[ℝ]` corresponds to taking
-- the first partial derivative
example : (∂₀[ℝ] fun (x : ℝ × ℝ) => x.1) 0 = 1 := by
simp [Pi.zero_def, lineDeriv]
```
This has already been discussed on Zulip [here](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Partial.20derivatives).
I've opened this PR as a draft in order to get preliminary feedback on the contents (e.g. is this appropriate for Mathlib?); the file contains some demos of the notation in action.
Co-authored-by: Eric Wieser
---
- [ ] depends on: #25425
[](https://gitpod.io/from-referrer/)
|
t-analysis
merge-conflict
blocked-by-other-PR
|
195/0 |
Mathlib.lean,Mathlib/Analysis/Calculus/PartialDerivatives/Notation.lean,Mathlib/LinearAlgebra/Basis/HasCanonicalBasis.lean |
3 |
16 |
['Paul-Lez', 'github-actions', 'leanprover-community-bot-assistant', 'lecopivo', 'mathlib4-dependent-issues-bot', 'ocfnash'] |
nobody |
40-1570 1 month ago |
40-1570 1 month ago |
0-0 0 seconds |
27510 |
chrisflav author:chrisflav |
feat(RingTheory/Height): height of ideal is height of preimage plus height in quotient |
If `S` has going-down over `R`, the height of a prime `P` lying over `p` equals the height of `p` plus the height of the image of `P` in `S / p S`.
Co-authored by: Sihan Su
Co-authored by: Yi Song
---
- [ ] depends on: #22300
- [ ] depends on: #27508
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
large-import
blocked-by-other-PR
|
192/1 |
Mathlib/Data/Finset/Card.lean,Mathlib/Data/Fintype/Card.lean,Mathlib/Logic/Function/Basic.lean,Mathlib/RingTheory/Ideal/GoingDown.lean,Mathlib/RingTheory/Ideal/Height.lean,Mathlib/RingTheory/Ideal/KrullsHeightTheorem.lean,Mathlib/RingTheory/Ideal/MinimalPrime/Basic.lean,Mathlib/RingTheory/Ideal/Over.lean,Mathlib/RingTheory/Ideal/Quotient/Operations.lean,Mathlib/RingTheory/Spectrum/Prime/RingHom.lean |
10 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
39-61402 1 month ago |
39-61402 1 month ago |
0-1531 25 minutes |
25143 |
chrisflav author:chrisflav |
feat(RingTheory): smooth algebras have smooth Noetherian models |
Co-authored by: Judith Ludwig
---
- [ ] depends on: #24794
- [ ] depends on: #25138
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
merge-conflict
blocked-by-other-PR
|
596/45 |
Mathlib.lean,Mathlib/Algebra/Algebra/Subalgebra/Basic.lean,Mathlib/Algebra/Algebra/Subalgebra/Tower.lean,Mathlib/Algebra/Algebra/Tower.lean,Mathlib/Algebra/MvPolynomial/Basic.lean,Mathlib/Algebra/MvPolynomial/Eval.lean,Mathlib/RingTheory/AlgebraicIndependent/Transcendental.lean,Mathlib/RingTheory/Extension/Presentation/Basic.lean,Mathlib/RingTheory/Extension/Presentation/Core.lean,Mathlib/RingTheory/FinitePresentation.lean,Mathlib/RingTheory/FiniteType.lean,Mathlib/RingTheory/Ideal/Cotangent.lean,Mathlib/RingTheory/Ideal/Maps.lean,Mathlib/RingTheory/Ideal/Quotient/Operations.lean,Mathlib/RingTheory/MvPolynomial/Homogeneous.lean,Mathlib/RingTheory/Smooth/Basic.lean,Mathlib/RingTheory/Smooth/Kaehler.lean,Mathlib/RingTheory/Smooth/NoetherianDescent.lean,Mathlib/RingTheory/Spectrum/Prime/ChevalleyComplexity.lean,Mathlib/RingTheory/TensorProduct/MvPolynomial.lean,Mathlib/RingTheory/Unramified/Basic.lean |
21 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
39-3763 1 month ago |
39-3763 1 month ago |
0-713 11 minutes |
22909 |
AntoineChambert-Loir author:AntoineChambert-Loir |
feat(RingTheory/Pure): pure submodules |
A submodule `N` of an `R`-module is *pure* if all maps `S ⊗[R] N → S ⊗[R] M`
deduced by base change from the injection of `N` into `M` are injective,
for all `R`-algebras `S`.
This is expressed by the class `Submodule.IsPure`.
For type theoretic reason, the definition of `Submodule.IsPure` only considers
algebras `S` in the same universe as `R`, but `Submodule.IsPure.baseChange_injective`
establishes the property for all universes.
* `Submodule.IsComplemented.isPure` : a complemented submodule is pure.
Co-authored with @mariainesdff
---
- [ ] depends on: #22898
- [ ] depends on: #22908
- [x] depends on: #22911
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
merge-conflict
blocked-by-other-PR
|
592/3 |
Mathlib.lean,Mathlib/Algebra/Algebra/Equiv.lean,Mathlib/RingTheory/Adjoin/FG.lean,Mathlib/RingTheory/Finiteness/Basic.lean,Mathlib/RingTheory/Finiteness/Cardinality.lean,Mathlib/RingTheory/Finiteness/Small.lean,Mathlib/RingTheory/Pure.lean,Mathlib/RingTheory/Spectrum/Prime/RingHom.lean,Mathlib/RingTheory/TensorProduct/Basic.lean,Mathlib/RingTheory/TensorProduct/DirectLimit/FG.lean,Mathlib/RingTheory/TensorProduct/DirectLimit/Small.lean |
11 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
39-3697 1 month ago |
39-3697 1 month ago |
0-1047 17 minutes |
22908 |
AntoineChambert-Loir author:AntoineChambert-Loir |
feat(RingTheory/Finiteness/Small): tensor product of the system of small submodules |
The directed limit of a tensor product for the directed system of small submodules.
Co-authored with @mariainesdff
---
- [ ] depends on: #22898
- [x] depends on: #22911
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
merge-conflict
blocked-by-other-PR
|
624/2 |
Mathlib.lean,Mathlib/RingTheory/Adjoin/FG.lean,Mathlib/RingTheory/Finiteness/Basic.lean,Mathlib/RingTheory/Finiteness/Cardinality.lean,Mathlib/RingTheory/Finiteness/Small.lean,Mathlib/RingTheory/Spectrum/Prime/RingHom.lean,Mathlib/RingTheory/TensorProduct/Basic.lean,Mathlib/RingTheory/TensorProduct/DirectLimit/FG.lean,Mathlib/RingTheory/TensorProduct/DirectLimit/Small.lean |
9 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
39-3649 1 month ago |
39-3649 1 month ago |
0-3552 59 minutes |
27978 |
smmercuri author:smmercuri |
feat: `InfinitePlace.Extension` API for extensions of infinite places. |
This PR continues the work from #24881.
Original PR: https://github.com/leanprover-community/mathlib4/pull/24881
---
- [ ] depends on: #27977 |
t-number-theory
blocked-by-other-PR
|
181/0 |
Mathlib/NumberTheory/NumberField/InfinitePlace/Embeddings.lean,Mathlib/NumberTheory/NumberField/InfinitePlace/Ramification.lean |
2 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
38-85187 1 month ago |
38-85188 1 month ago |
0-421 7 minutes |
27971 |
smmercuri author:smmercuri |
feat: weak approximation theorems for infinite places of a number field |
This PR continues the work from #22153.
Original PR: https://github.com/leanprover-community/mathlib4/pull/22153
---
- [ ] depends on: #27970 |
t-algebra
t-number-theory
blocked-by-other-PR
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 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'smmercuri'] |
nobody |
38-83687 1 month ago |
38-83687 1 month ago |
0-2675 44 minutes |
26377 |
Whysoserioushah author:Whysoserioushah |
feat(Mathlib/RingTheory/SimpleRing/TensorProduct): Tensor product of a simple algebra and a central simple algebra is simple |
co-authored-by: @jjaassoonn
---
- [ ] depends on: #26368
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
merge-conflict
blocked-by-other-PR
|
423/0 |
Mathlib.lean,Mathlib/RingTheory/SimpleRing/TensorProduct.lean,Mathlib/RingTheory/TwoSidedIdeal/SpanAsSum.lean |
3 |
15 |
['Whysoserioushah', 'eric-wieser', 'github-actions', 'kckennylau', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
38-77452 1 month ago |
38-77453 1 month ago |
0-2337 38 minutes |
27493 |
themathqueen author:themathqueen |
feat(RingTheory/Coalgebra): define Frobenius algebra |
A Frobenius algebra `A` has the structure of both an algebra and a coalgebra such that:
`(mul ⊗ id) ∘ assoc.symm ∘ (id ⊗ comul) = comul ∘ mul = (id ⊗ mul) ∘ assoc ∘ (comul ⊗ id)`.
In diagrams this law looks like:

It suffices to show that
`(mul ⊗ id) ∘ assoc.symm ∘ (id ⊗ comul) = (id ⊗ mul) ∘ assoc ∘ (comul ⊗ id)`
(the proof of this is ugly).
---
- [ ] depends on: #27567
- [x] depends on: #27569
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
blocked-by-other-PR
|
224/0 |
Mathlib.lean,Mathlib/LinearAlgebra/TensorProduct/Tower.lean,Mathlib/RingTheory/Coalgebra/Frobenius.lean |
3 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
38-68622 1 month ago |
39-61232 1 month ago |
2-700 2 days |
28001 |
daefigueroa author:daefigueroa |
feat(Dynamics): add results on topologically transitive flows |
We define topological transitivity for a flow and show that a factor of a topologically transitive flow is topologically transitive.
---
This contribution was created as part of the Utrecht Summerschool "Formalizing Mathematics in Lean" in July 2025.
- [ ] depends on: #28000
[](https://gitpod.io/from-referrer/) |
new-contributor
t-dynamics
blocked-by-other-PR
|
68/3 |
Mathlib.lean,Mathlib/Dynamics/Flow.lean,Mathlib/Dynamics/Transitive.lean |
3 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
38-47985 1 month ago |
38-47985 1 month ago |
0-89 1 minute |
14089 |
callesonne author:callesonne |
feat(Bicategory/Functorbicategory): define bicategory of pseudofunctors |
This PR contains a definition of the bicategory of pseudofunctors, in the file `Bicategory/FunctorBicategory/Pseudo.lean`. It also moves the file `Bicategory/Functorbicategory.lean` to `Bicategory/FunctorBicategory/Oplax.lean`.
---
- [x] depends on: #14028
- [x] depends on: #18250
- [x] depends on: #18252
- [x] depends on: #18253
- [ ] depends on: #18254
[](https://gitpod.io/from-referrer/)
|
t-category-theory
merge-conflict
blocked-by-other-PR
|
385/70 |
Mathlib.lean,Mathlib/CategoryTheory/Bicategory/FunctorBicategory/Oplax.lean,Mathlib/CategoryTheory/Bicategory/FunctorBicategory/Pseudo.lean,Mathlib/CategoryTheory/Bicategory/Modification/Oplax.lean,Mathlib/CategoryTheory/Bicategory/Modification/Pseudo.lean,Mathlib/CategoryTheory/Bicategory/NaturalTransformation/Oplax.lean,Mathlib/CategoryTheory/Bicategory/NaturalTransformation/Pseudo.lean |
7 |
6 |
['callesonne', 'github-actions', 'leanprover-community-bot-assistant', 'leanprover-community-mathlib4-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
38-35945 1 month ago |
38-35946 1 month ago |
9-2320 9 days |
26578 |
robin-carlier author:robin-carlier |
feat(CategoryTheory/Limits/Pullbacks/Categorical/CatCospanTransform): adjunctions of categorical cospans |
We build upon the bicategory-like structure developed in #26447 and #26412 to define the notion of adjunctions of categorical cospans. This is a structure encoding the data of two `CatCospanTransform`s, along with the usual unit and counit morphisms as part of the data, satisfying the usual left and right triangle identities. We provide basic API for these, such as extracting adjunctions between individual components. We also provide a proof that the notion satisfies a "coherence": with our chosen constructor, the forward direction of the structure `CatCommSq` on the left adjoints correspond to the inverse of the square for the right adjoints through `mateEquiv`.
These adjunctions will be used as a substrate for defining equivalences of categorical cospans in a future PR: such an equivalence will be a structure extending a `CatCospanAdjunction` with isomorphisms data on the unit and co-unit (we will however provide alternative constructors in sync with the constructor for equivalences of categories).
---
- [x] depends on: #26447
- [ ] depends on: #26547
[](https://gitpod.io/from-referrer/)
|
large-import
t-category-theory
blocked-by-other-PR
|
205/0 |
Mathlib/CategoryTheory/Limits/Shapes/Pullback/Categorical/CatCospanTransform.lean |
1 |
4 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
38-11022 1 month ago |
38-11041 1 month ago |
0-625 10 minutes |
26579 |
robin-carlier author:robin-carlier |
feat(CategoryTheory/Limits/Pullbacks/Categorical/CatCospanTransform): equivalences of categorical cospans |
Building on the notion of adjunctions of categorical cospans, we define equivalences of categorical cospans as a structure extending that of an adjunction, with the extra data of a chosen inverse of the unit and counit morphisms.
To mirror the design for usual equivalences of categories, we provide an alternative constructor that requires the forward and
inverse direction of the equivalence, as well as unit and counits already as isomorphisms, and only a proof of the left triangle identity.
Finally, we also provide a third constructor that builds such an equivalence out of the data of 3 component equivalences of categories, as well as chosen `CatCommSq` on the functors of the these equivalences.
This notion of equivalence of categorical cospans is intended to encode the required data to show the full equivalence invariance of the categorical pullback defined in #26366.
---
- [ ] depends on: #26578
[](https://gitpod.io/from-referrer/)
|
large-import
t-category-theory
blocked-by-other-PR
|
438/0 |
Mathlib/CategoryTheory/Limits/Shapes/Pullback/Categorical/CatCospanTransform.lean |
1 |
4 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
38-10924 1 month ago |
38-10945 1 month ago |
0-838 13 minutes |
27214 |
robin-carlier author:robin-carlier |
feat(CategoryTheory/Limits/Shapes/Pullback/Categorical): Categorical pullback squares |
In this PR, we give the definition and first basic properties of categorical pullback squares.
Using our previous work on `CategoricalPullback`, we define a typeclass `CatPullbackSquare T L R B` that asserts that a given `CatCommSq T L R B` is a "pullback square": this is the data of a chosen adjoint equivalence to the canonical functor from the top left corner of the square to the categorical pulback of its leg. Using this equivalence, be derive a universal property for functors from `X`with values in the top left corner of the square: they are equivalent to `CatCommSqOver R B X`, the category of categorical commutative squares over the cospan `R, B` with top left corner `X`.
We prove some coherence result for this equivalence, most notably an isomorphism that, given `S : CatCommSqOver R B X`, bundles the two commutative triangles formed by the induced functor, and the coherence between the squares that these isomorphisms satisfy: this is conveniently bundled in the data of a single isomorphisms of `CatCommSqOver R B X`.
Finally, we provide a `Prop`-class `IsCatPullbackSquare` that merely asserts the existence (via `Nonempty`) of the relevant data: we show that it is tautotogically equivalent to the propopsition that the canonical functor to the categorical pullback is an equivalence.
---
- [ ] depends on: #26679
[](https://gitpod.io/from-referrer/)
|
t-category-theory
blocked-by-other-PR
|
786/1 |
Mathlib.lean,Mathlib/CategoryTheory/Limits/Shapes/Pullback/Categorical/Basic.lean,Mathlib/CategoryTheory/Limits/Shapes/Pullback/Categorical/Square.lean |
3 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
38-10069 1 month ago |
50-70475 1 month ago |
0-1477 24 minutes |
27391 |
robin-carlier author:robin-carlier |
feat(CategoryTheory/Limits/Shapes/Pullback/Categorical): pseudofunctoriality structure of categorical pullback squares |
Using pseudofunctoriality of the construction `CatCommSqOver`, we show that categorical pullback squares have pseudofunctorial-like structures: given a `CatCommSq T L R B` and a `CatPullbackSq T' L' R' B'`, and a `CatCospanTransform R B R' B'`, there is a
functor `CatPullbackSq.functorOfTransform` between the top left corners of the two squares. We give `CatCommSq` instances that relates this functor with other constructions such as `CatCommSqOver.transform`.
Similarly, we construct `CatPullbackSq.functorOfTransform₂`, that maps morphisms of `CatCospanTransforms` to natural transformations. Finally, we show that `functorOfTransform` respects identities and compositions.
We do not yet prove that all of this data satisfies all the expected properties of pseudofunctors: this will be the content of a follow-up PR.
---
- [ ] depends on: #27214
[](https://gitpod.io/from-referrer/)
|
t-category-theory
blocked-by-other-PR
|
1090/1 |
Mathlib.lean,Mathlib/CategoryTheory/Limits/Shapes/Pullback/Categorical/Basic.lean,Mathlib/CategoryTheory/Limits/Shapes/Pullback/Categorical/Square.lean |
3 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
38-10040 1 month ago |
48-69728 1 month ago |
0-264 4 minutes |
27432 |
robin-carlier author:robin-carlier |
feat(CategoryTheory/Limits/Shapes/Pullback/Categorical): pseudofunctoriality of categorical pulback squares |
In this PR, we show that the "unbundled pseudofunctor" data constructed in #27391 satisfy the axioms of an actual "unbundled pseudo-functor". This is intended to give all the required coherence for a formal bicategory-like proof of the fact that `CatCospanAdjunction`s from #26578 (resp. `CatCospanEquivalence`s from #26579) promote to adjunctions (resp. equivalences) between the top left corners of categorical pullback squares.
---
- [ ] depends on: #27391
[](https://gitpod.io/from-referrer/)
|
t-category-theory
blocked-by-other-PR
|
1244/1 |
Mathlib.lean,Mathlib/CategoryTheory/Limits/Shapes/Pullback/Categorical/Basic.lean,Mathlib/CategoryTheory/Limits/Shapes/Pullback/Categorical/Square.lean |
3 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
38-9976 1 month ago |
48-69707 1 month ago |
0-1056 17 minutes |
27481 |
robin-carlier author:robin-carlier |
feat(CategoryTheory/Limits/Shapes/Pullback/Categorical): adjunctions and equivalences of categorical pullback squares |
We show that a `CatCospanAdjunction` (resp `CatCospanEquivalence`) induces adjunctions (resp. equivalences) of the categories that sit at the top left corners of categorical pullback squares via the pseudofunctoriality proved in #27432. Thanks to the lemmas that proves that categorical pullback squares are fully pseudofunctorial, the proof is purely formal ("a pseudofunctor maps adjunctions (resp. equivalences) to adjunctions (resp. equivalences)"), rather than being a painful computation for the triangle equalities.
In particular, the results here show that two categorical pullback squares with equivalent "underlying categorical cospan" are equivalent, which realizes the equivalence-invariance of the notion of categorical pullbacks.
We do not yet show that a (not-necessarily pullback) `CatCommSq T L R B` equivalent to a `CatPullbackSquare T' L' R' B'` via a
`CatCospanEquivalence R B R' B'` is also a `CatPullbackSquare`: this will be the content of a follow-up PR.
---
- [ ] depends on: #27432
- [ ] depends on: #26579
[](https://gitpod.io/from-referrer/)
|
large-import
t-category-theory
blocked-by-other-PR
|
1829/1 |
Mathlib.lean,Mathlib/CategoryTheory/Limits/Shapes/Pullback/Categorical/Basic.lean,Mathlib/CategoryTheory/Limits/Shapes/Pullback/Categorical/CatCospanTransform.lean,Mathlib/CategoryTheory/Limits/Shapes/Pullback/Categorical/Square.lean |
4 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
38-9864 1 month ago |
49-64968 1 month ago |
0-49 49 seconds |
27686 |
robin-carlier author:robin-carlier |
feat(CategoryTheory/Limits/Shapes/Pullback/Categorical/Square): more API for `CatPullbackSquare` |
In this PR, we provide more API around the notion of categorical pullback squares. Having established the pseudofunctoriality of the notion in #27432, we characterize the behaviour of the equivalence
`CatPullbackSquare.functorEquiv (π₁ R B) (π₂ R B) R B X : X ⥤ R ⊡ B ≌ CatCommSqOver R B X` via various (d)simp lemmas. This ports all the pseudofunctoriality and equivalence-invariance results of `CatPullbackSquare` to `CategoricalPullback`.
We also show this equivalence is isomorphic to the one from `CategoricalPullback.functorEquiv`.
Unfortunately, this small duplication is necessary, as `CatPullbackSquare.functorEquiv` is bulit using `CategoricalPullback.functorEquiv`. The equivalence `CategoricalPullback.functorEquiv` is now an implementation detail, the idiomatic way is to use `CatPullbackSquare.functorEquiv`; docstrings are updated accordingly.
This deprecates some constructions and lemmas for `CategoricalPullback`: they are now special case of the API that is available for any categorical pullback square.
---
- [ ] depends on: #27481
[](https://gitpod.io/from-referrer/)
|
large-import
t-category-theory
blocked-by-other-PR
|
2245/74 |
Mathlib.lean,Mathlib/CategoryTheory/Limits/Shapes/Pullback/Categorical/Basic.lean,Mathlib/CategoryTheory/Limits/Shapes/Pullback/Categorical/CatCospanTransform.lean,Mathlib/CategoryTheory/Limits/Shapes/Pullback/Categorical/Square.lean |
4 |
n/a |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
38-9561 1 month ago |
unknown |
unknown |
27688 |
robin-carlier author:robin-carlier |
feat(CategoryTheory/Limits/Shapes/Pullback/Categorical): coherence statement for `CatPullbackSquare.inverse` |
This PR records a "coherence" statement for `CatPullbackSquares`: it bridges the gap between the user-provided `inverse` field of the `CatPullbackSquare` structure, and the other way one can deduce an equivalence between the top left corner of the square and a categorical pullback (via the pseudofunctoriality of categorical pullback squares induced by the identity `CatCospanTransform`). We show the two possible natural isomorphisms on the inverses of the equivalences are in fact the same (hence the term "coherence").
---
- [ ] depends on: #27686
[](https://gitpod.io/from-referrer/)
|
large-import
t-category-theory
blocked-by-other-PR
|
2351/74 |
Mathlib.lean,Mathlib/CategoryTheory/Limits/Shapes/Pullback/Categorical/Basic.lean,Mathlib/CategoryTheory/Limits/Shapes/Pullback/Categorical/CatCospanTransform.lean,Mathlib/CategoryTheory/Limits/Shapes/Pullback/Categorical/Square.lean |
4 |
n/a |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
38-9241 1 month ago |
unknown |
unknown |
27687 |
robin-carlier author:robin-carlier |
feat(CategoryTheory/Limits/Shapes/Pullback/Categorical): squares equivalent to a `CatPullbackSquare` |
We provide the last remaining piece of the "equivalence-invariance" of categorical pullback squares: given a `CatCommSq (T : C₁ ⥤ _) L R B`, a `CatPullbackSquare (T' : D₁ ⥤ _) L' R' B'`, a `ψ : CatCospanEquivalence R B R' B'` and an equivalence `C₁ ≌ D₁` that identifies to the functor induced by `ψ`, the `CatCommSq T L R B` can be promoted to a `CatPullbackSquare T L R B'`.
In other words: a `CatCommSq` that is equivalent to a `CatPullbackSquare` is a `CatPullbackSquare`.
---
- [ ] depends on: #27686
[](https://gitpod.io/from-referrer/)
|
large-import
t-category-theory
blocked-by-other-PR
|
2318/74 |
Mathlib.lean,Mathlib/CategoryTheory/Limits/Shapes/Pullback/Categorical/Basic.lean,Mathlib/CategoryTheory/Limits/Shapes/Pullback/Categorical/CatCospanTransform.lean,Mathlib/CategoryTheory/Limits/Shapes/Pullback/Categorical/Square.lean |
4 |
n/a |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
38-9184 1 month ago |
unknown |
unknown |
27689 |
robin-carlier author:robin-carlier |
feat(CategoryTheory/Limits/Shapes/Pullback/Categorical): horizontal pasting calculus for `CatPullbackSquare` |
Given two categorical commutative squares that can be horizontally pasted, we prove that if the rightmost square is a `CatPullbackSquare`, then the leftmost square is a `CatPullbackSquare` if and only if the horizontal composition of the squares is a `CatPullbackSquare`. This generalizes to `CatPullbackSquare` the well-known "pasting calculus" for pullback squares in a category.
The statement is made available both in terms of the `Type`-class `CatPullbackSquare`, and in terms of the `Prop`-class `IsCatPullbackSquare`.
---
- [ ] depends on: #27686
[](https://gitpod.io/from-referrer/)
|
large-import
t-category-theory
blocked-by-other-PR
|
2562/74 |
Mathlib.lean,Mathlib/CategoryTheory/Limits/Shapes/Pullback/Categorical/Basic.lean,Mathlib/CategoryTheory/Limits/Shapes/Pullback/Categorical/CatCospanTransform.lean,Mathlib/CategoryTheory/Limits/Shapes/Pullback/Categorical/Pasting.lean,Mathlib/CategoryTheory/Limits/Shapes/Pullback/Categorical/Square.lean |
5 |
n/a |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
38-9131 1 month ago |
unknown |
unknown |
27690 |
robin-carlier author:robin-carlier |
feat(CategoryTheory/Limits/Shapes/Pullback/Categorical): vertical pasting calculus for `CatPullbackSquare` |
We mirror the constructions from #27689 to construct the vertical pasting calculus of `CatPullbackSquares`: given two vertically composable `CatCommSq` such that the bottom one is a `CatPullbackSquare`, the top square is a `CatPullbackSquare` if and only if the vertical composition (the "outer" square) is a `CatPullbackSquare`.
---
- [ ] depends on: #27689
[](https://gitpod.io/from-referrer/)
|
large-import
t-category-theory
blocked-by-other-PR
|
2841/74 |
Mathlib.lean,Mathlib/CategoryTheory/Limits/Shapes/Pullback/Categorical/Basic.lean,Mathlib/CategoryTheory/Limits/Shapes/Pullback/Categorical/CatCospanTransform.lean,Mathlib/CategoryTheory/Limits/Shapes/Pullback/Categorical/Pasting.lean,Mathlib/CategoryTheory/Limits/Shapes/Pullback/Categorical/Square.lean |
5 |
n/a |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
38-9076 1 month ago |
unknown |
unknown |
27740 |
robin-carlier author:robin-carlier |
feat(CategoryTheory/Limits/Shapes/Pullback/Categorical): pasting calculus for `CategoricalPullback` |
Specialize the pasting calculus for categorical pullback squares to `CategoricalPullback̀` by providing equivalences of categories `R ⊡ (B₁ ⋙ B₂) ≌ (π₂ R B₂) ⊡ B₁` and `(R₁ ⋙ R₂) ⊡ B ≌ R₁ ⊡ (π₁ R₂ B)`. The `@[simps!]` attribute works wonderfully on these equivalences so that their component all have the expected (d)simp lemmas.
---
- [ ] depends on: #27690
[](https://gitpod.io/from-referrer/)
|
large-import
t-category-theory
blocked-by-other-PR
|
2872/75 |
Mathlib.lean,Mathlib/CategoryTheory/Limits/Shapes/Pullback/Categorical/Basic.lean,Mathlib/CategoryTheory/Limits/Shapes/Pullback/Categorical/CatCospanTransform.lean,Mathlib/CategoryTheory/Limits/Shapes/Pullback/Categorical/Pasting.lean,Mathlib/CategoryTheory/Limits/Shapes/Pullback/Categorical/Square.lean |
5 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
38-9028 1 month ago |
38-9051 1 month ago |
0-1017 16 minutes |
27982 |
ShreckYe author:ShreckYe |
chore(Data/Nat/GCD): use `Nat.Prime.dvd_or_dvd` from #27981 in `Nat.Prime.dvd_or_dvd_of_dvd_lcm` from #27963 to simplify the proof a bit |
- [ ] depends on: #27963
- [ ] depends on: #27981 |
large-import
new-contributor
blocked-by-other-PR
|
102/2 |
Mathlib/Algebra/GCDMonoid/Basic.lean,Mathlib/Data/Nat/GCD/Basic.lean,Mathlib/Data/Nat/Prime/Defs.lean |
3 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
37-8373 1 month ago |
38-81459 1 month ago |
0-1834 30 minutes |
25825 |
yuma-mizuno author:yuma-mizuno |
feat(CategoryTheory/Bicategory): define lax transformations between oplax functors |
and also define oplax transformations between lax functors.
- [ ] depends on: #25779
---
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #25672.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/25672* |
large-import
t-category-theory
blocked-by-other-PR
|
431/10 |
Mathlib.lean,Mathlib/CategoryTheory/Bicategory/NaturalTransformation/Lax.lean,Mathlib/CategoryTheory/Bicategory/NaturalTransformation/Oplax.lean,scripts/noshake.json |
4 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
37-1993 1 month ago |
37-2012 1 month ago |
0-1 1 second |
26668 |
mariainesdff author:mariainesdff |
feat(Analysis/Normed/Unbundled/SpectralNorm): add API |
Co-authored-by: @faenuccio
---
- [ ] depends on: #26667
[](https://gitpod.io/from-referrer/)
|
t-analysis
t-number-theory
merge-conflict
blocked-by-other-PR
|
149/11 |
Mathlib/Algebra/Polynomial/Lifts.lean,Mathlib/Analysis/Normed/Unbundled/SpectralNorm.lean,Mathlib/FieldTheory/SplittingField/IsSplittingField.lean |
3 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
35-71645 1 month ago |
35-71646 1 month ago |
0-1623 27 minutes |
28152 |
Sebi-Kumar author:Sebi-Kumar |
feat(AlgebraicTopology): characterize simply connectedness in terms of loops |
Show that a space is simply connected if and only if all loops within that space are homotopic to the constant loop. To be used in a proof that the `n`-sphere is simply connected for `n > 1`.
---
This code was written at the University of Western Ontario as a part of the Fields Undergraduate Summer Research Program under the supervision of Chris Kapulkin and Daniel Carranza.
- [ ] depends on: #28126
[](https://gitpod.io/from-referrer/)
|
t-algebraic-topology
new-contributor
blocked-by-other-PR
|
37/5 |
Mathlib/AlgebraicTopology/FundamentalGroupoid/Basic.lean,Mathlib/AlgebraicTopology/FundamentalGroupoid/SimplyConnected.lean |
2 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
34-68126 1 month ago |
34-68127 1 month ago |
0-2854 47 minutes |
28208 |
Sebi-Kumar author:Sebi-Kumar |
feat(Topology): add the definition `foldTrans` to concatenate finite sequences of paths |
Add `foldTrans`, which folds the function `Path.trans` across a sequence of paths with compatible endpoints, corresponding to the concatenation of a finite sequence of paths. This is implemented with `Fin.dfoldl` from the Batteries library. Prove basic properties about `foldTrans` (i.e., how it behaves with respect to `Path.refl`, `Path.subpath`, and homotopies).
---
To provide additional context, I am new to contributing to Mathlib, and I am doing so as a part of the Fields Undergraduate Summer Research Program at the University of Western Ontario under the supervision of Chris Kapulkin and Daniel Carranza. My goal is to prove that the `n`-sphere is simply connected for `n > 1`, following the proof from Hatcher's "Algebraic Topology."
- [ ] depends on: #27261
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-topology
blocked-by-other-PR
|
259/0 |
Mathlib.lean,Mathlib/Topology/FoldTrans.lean,Mathlib/Topology/Subpath.lean |
3 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
33-37766 1 month ago |
33-37767 1 month ago |
0-2340 39 minutes |
27100 |
staroperator author:staroperator |
feat(ModelTheory): Presburger definability and semilinear sets |
This PR defines [semilinear sets](https://en.wikipedia.org/wiki/Semilinear_set) and formalizes their equivalence with Presburger definabilty. As an application of this result, we prove that the graph of multiplication is not Presburger definable in ℕ.
---
- [x] depends on: #26896
- [x] depends on: #27081
- [x] depends on: #27087
- [ ] depends on: #27789
---
[](https://gitpod.io/from-referrer/)
|
t-logic
merge-conflict
blocked-by-other-PR
|
1667/7 |
Mathlib.lean,Mathlib/Algebra/Group/Submonoid/Defs.lean,Mathlib/Algebra/Module/Submodule/Defs.lean,Mathlib/GroupTheory/Finiteness.lean,Mathlib/LinearAlgebra/LinearIndependent/Defs.lean,Mathlib/ModelTheory/Arithmetic/Presburger/Definability.lean,Mathlib/ModelTheory/Arithmetic/Presburger/Semilinear/Basic.lean,Mathlib/ModelTheory/Arithmetic/Presburger/Semilinear/Defs.lean,Mathlib/ModelTheory/Arithmetic/Presburger/Semilinear/Nat.lean,Mathlib/Order/WellFoundedSet.lean,Mathlib/RingTheory/Finiteness/Cardinality.lean,docs/references.bib |
12 |
6 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
32-80960 1 month ago |
32-80961 1 month ago |
0-1811 30 minutes |
28067 |
grunweg author:grunweg |
Docstring enumerations |
Tracking PR; to be split. Audit all ocurrences of `^ \S`; exhaustive.
---
- [x] depends on: #28068
- [x] depends on: #28069
- [ ] depends on: #28070
- [x] depends on: #28118
[](https://gitpod.io/from-referrer/)
|
blocked-by-other-PR |
264/263 |
Archive/Wiedijk100Theorems/SumOfPrimeReciprocalsDiverges.lean,Mathlib/Algebra/Algebra/Defs.lean,Mathlib/Algebra/BrauerGroup/Defs.lean,Mathlib/Algebra/Module/LinearMap/Polynomial.lean,Mathlib/CategoryTheory/Abelian/NonPreadditive.lean,Mathlib/CategoryTheory/EqToHom.lean,Mathlib/CategoryTheory/Filtered/Basic.lean,Mathlib/CategoryTheory/Limits/Final.lean,Mathlib/CategoryTheory/Limits/Pi.lean,Mathlib/CategoryTheory/Monoidal/Center.lean,Mathlib/CategoryTheory/Sites/Grothendieck.lean,Mathlib/CategoryTheory/Sites/Pretopology.lean,Mathlib/Condensed/Discrete/Characterization.lean,Mathlib/FieldTheory/ChevalleyWarning.lean,Mathlib/GroupTheory/MonoidLocalization/Basic.lean,Mathlib/LinearAlgebra/CliffordAlgebra/Basic.lean,Mathlib/LinearAlgebra/Multilinear/Basic.lean,Mathlib/LinearAlgebra/RootSystem/GeckConstruction/Basic.lean,Mathlib/MeasureTheory/Integral/Bochner/Basic.lean,Mathlib/MeasureTheory/Measure/MeasureSpace.lean,Mathlib/MeasureTheory/Measure/MeasureSpaceDef.lean,Mathlib/MeasureTheory/OuterMeasure/Basic.lean,Mathlib/MeasureTheory/OuterMeasure/Defs.lean,Mathlib/NumberTheory/FLT/Basic.lean,Mathlib/NumberTheory/LSeries/PrimesInAP.lean,Mathlib/RingTheory/Grassmannian.lean,Mathlib/RingTheory/Localization/Basic.lean,Mathlib/RingTheory/Localization/Defs.lean,Mathlib/RingTheory/WittVector/Teichmuller.lean,Mathlib/Tactic/Bound.lean,Mathlib/Tactic/Bound/Attribute.lean,Mathlib/Tactic/ENatToNat.lean,Mathlib/Tactic/FBinop.lean,Mathlib/Tactic/IntervalCases.lean,Mathlib/Tactic/TermCongr.lean,Mathlib/Util/Notation3.lean,Mathlib/Util/Superscript.lean,docs/Conv/Guide.lean |
38 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
32-75573 1 month ago |
37-8386 1 month ago |
0-2904 48 minutes |
28243 |
robin-carlier author:robin-carlier |
chore(CategoryTheory/Bicategory): move some `eqToHom` lemmas |
The file `CategoryTheory/Bicategory/EqToHom.lean` introduced in #28242 is a more suitable hom for the lemmas `CategoryTheory.Bicategory.whiskerLeft_eqToHom` and `CategoryTheory.Bicategory.eqToHom_whiskerRight` than the current `CategoryTheory/Bicategory/Strict.lean`. We move these lemmas to the new file, and make `CategoryTheory/Bicategory/Strict` import these lemmas.
---
- [ ] depends on: #28242
[](https://gitpod.io/from-referrer/)
|
t-category-theory
blocked-by-other-PR
|
165/23 |
Mathlib.lean,Mathlib/CategoryTheory/Bicategory/EqToHom.lean,Mathlib/CategoryTheory/Bicategory/Strict.lean,Mathlib/CategoryTheory/EqToHom.lean,scripts/noshake.json |
5 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'robin-carlier'] |
nobody |
32-67419 1 month ago |
32-67419 1 month ago |
0-3342 55 minutes |
27626 |
EtienneC30 author:EtienneC30 |
chore: turn covarianceBilin into a ContinuousBilinForm |
From BrownianMotion
---
- [ ] depends on: #26315
[](https://gitpod.io/from-referrer/)
|
large-import
t-measure-probability
merge-conflict
blocked-by-other-PR
|
275/2 |
Mathlib.lean,Mathlib/Analysis/NormedSpace/ContinuousBilinForm.lean,Mathlib/LinearAlgebra/BilinearForm/IsPosSemidef.lean,Mathlib/LinearAlgebra/Matrix/BilinearForm.lean,Mathlib/LinearAlgebra/Matrix/Hermitian.lean,Mathlib/Probability/Moments/CovarianceBilin.lean |
6 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
32-21438 1 month ago |
32-21438 1 month ago |
0-384 6 minutes |
27645 |
bjornsolheim author:bjornsolheim |
feat(Geometry/Convex/Cone): add pointed cone tensor products |
Define the minimal and maximal tensor product of pointed cones.
Prove that the minimal tensor product is less than or equal to the maximal tensor product.
---
- [ ] depends on: #25292
- [ ] depends on: #27578
[](https://gitpod.io/from-referrer/)
|
t-convex-geometry
new-contributor
blocked-by-other-PR
|
316/0 |
Mathlib.lean,Mathlib/Geometry/Convex/Cone/ConicalHull.lean,Mathlib/Geometry/Convex/Cone/TensorProduct.lean |
3 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
31-52309 1 month ago |
31-55958 1 month ago |
0-1828 30 minutes |
28328 |
pechersky author:pechersky |
chore(Topology/Valued): golf using local finite order of WithZeroTopology |
have to juggle in a version of `mrangeRestrict`
which works on valuations,
and also juggle the scoped topology over
the subtype topology
---
[](https://gitpod.io/from-referrer/)
- [ ] depends on: #28325 |
large-import
t-algebra
t-topology
t-number-theory
blocked-by-other-PR
label:t-algebra$ |
187/88 |
Mathlib/Topology/Algebra/GroupWithZero.lean,Mathlib/Topology/Algebra/Valued/LocallyCompact.lean,Mathlib/Topology/Algebra/WithZeroTopology.lean,Mathlib/Topology/Compactness/Compact.lean |
4 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
31-15573 1 month ago |
31-15574 1 month ago |
0-1600 26 minutes |
26457 |
AntoineChambert-Loir author:AntoineChambert-Loir |
feat(Mathlib/GroupTheory/Perm/MaximalSubgroups): maximal subgroups of the permutation group |
* `Equiv.Perm.isCoatom_stabilizer`: when `s : Set α` is not empty, nor its complementary subset, and if the cardinality of `s` is not half of that of `α`, then `MulAction.stabilizer (Equiv.Perm α) s` is a maximal subgroup of the symmetric group `Equiv.Perm α`.
This is the *intransitive case* of the O'Nan-Scott classification.
## TODO
* Appplication to primitivity of the action of `Equiv.Perm α` on finite combinations of `α`.
* Finish the classification
---
- [ ] depends on: #26282
- [x] depends on: #26281
- [x] depends on: #26280
- [x] depends on: #26279
[](https://gitpod.io/from-referrer/)
|
t-group-theory
large-import
blocked-by-other-PR
|
1563/137 |
Mathlib.lean,Mathlib/Data/Set/Card.lean,Mathlib/GroupTheory/GroupAction/Jordan.lean,Mathlib/GroupTheory/GroupAction/MultiplePrimitivity.lean,Mathlib/GroupTheory/GroupAction/MultipleTransitivity.lean,Mathlib/GroupTheory/GroupAction/Primitive.lean,Mathlib/GroupTheory/GroupAction/SubMulAction/OfFixingSubgroup.lean,Mathlib/GroupTheory/GroupAction/SubMulAction/OfStabilizer.lean,Mathlib/GroupTheory/Perm/Cycle/Basic.lean,Mathlib/GroupTheory/Perm/Cycle/Type.lean,Mathlib/GroupTheory/Perm/MaximalSubgroups.lean,Mathlib/SetTheory/Cardinal/Embedding.lean,docs/references.bib |
13 |
n/a |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
31-587 1 month ago |
unknown |
unknown |
23915 |
joelriou author:joelriou |
feat(CategoryTheory): deriving functors using a right derivability structure |
We develop the API for derived functors following the existence theorem obtained in #26374. If `Φ` is a localizer morphism, we introduce a predicate `Φ.Derives F` for a functor `F` saying that `Φ.functor ⋙ F` inverts the given class of morphisms, and in case `Φ` is a right derivability structure, we show that `F` admits a right derived functor, and we obtain a recognition lemma for this derived functor.
(In the future, this will be applied to the injective/projective/flat derivability structures.)
---
- [ ] depends on: #26374
- [ ] depends on: #22474
- [ ] depends on: #26036
[](https://gitpod.io/from-referrer/)
|
t-category-theory
merge-conflict
blocked-by-other-PR
WIP
|
599/10 |
Mathlib.lean,Mathlib/CategoryTheory/Functor/Derived/PointwiseRightDerived.lean,Mathlib/CategoryTheory/Functor/Derived/RightDerived.lean,Mathlib/CategoryTheory/Functor/KanExtension/Pointwise.lean,Mathlib/CategoryTheory/Iso.lean,Mathlib/CategoryTheory/Limits/Final.lean,Mathlib/CategoryTheory/Limits/HasLimits.lean,Mathlib/CategoryTheory/Limits/Opposites.lean,Mathlib/CategoryTheory/Limits/Shapes/Products.lean,Mathlib/CategoryTheory/Localization/DerivabilityStructure/Basic.lean,Mathlib/CategoryTheory/Localization/DerivabilityStructure/Derives.lean,Mathlib/CategoryTheory/Localization/DerivabilityStructure/PointwiseRightDerived.lean |
12 |
4 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
30-81267 30 days ago |
124-49791 4 months ago |
0-0 0 seconds |
27673 |
b-reinke author:b-reinke |
feat(GroupTheory/FreeGroup): add cyclic reduction of words |
This PR adds the definition of `reduceCyclically`. This function produces a subword of a word `w` by cancelling the first and last letters of `w` as long as possible. If `w` is reduced, the resulting word will be cyclically reduced.
It is a part of a series of PR on the theory of cyclically reduced words.
Upstreamed from the [EquationalTheories](https://github.com/teorth/equational_theories) project.
- [ ] depends on: #25966
- [ ] depends on: #27672
---
[](https://gitpod.io/from-referrer/)
|
t-group-theory
merge-conflict
blocked-by-other-PR
|
235/0 |
Mathlib.lean,Mathlib/GroupTheory/FreeGroup/Basic.lean,Mathlib/GroupTheory/FreeGroup/CyclicallyReduced.lean,Mathlib/GroupTheory/FreeGroup/Reduce.lean |
4 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
30-65364 30 days ago |
30-65365 30 days ago |
0-1172 19 minutes |
27678 |
b-reinke author:b-reinke |
feat(GroupTheory/FreeGroup): reduction theorem for powers |
This PR adds the theorem `reduce_flatten_replicate`, it describes the reduction of a power of a reduced word in terms of its cyclic reduction.
It is a part of a series of PR on the theory of cyclically reduced words.
Upstreamed from the [EquationalTheories](https://github.com/teorth/equational_theories) project.
- [ ] depends on: #25966
- [ ] depends on: #27672
- [ ] depends on: #27673
---
[](https://gitpod.io/from-referrer/)
|
t-group-theory
merge-conflict
blocked-by-other-PR
|
286/0 |
Mathlib.lean,Mathlib/GroupTheory/FreeGroup/Basic.lean,Mathlib/GroupTheory/FreeGroup/CyclicallyReduced.lean,Mathlib/GroupTheory/FreeGroup/Reduce.lean |
4 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
30-65363 30 days ago |
30-65364 30 days ago |
0-19 19 seconds |
27679 |
b-reinke author:b-reinke |
feat(GroupTheory/FreeGroup): add pow_left_inj |
This PR shows that taking n-th powers is an injective function on the free group, using the theory of cyclical reduction.
It is the last part of a series of PR on the theory of cyclically reduced words, that were split from #22639.
Upstreamed from the [EquationalTheories](https://github.com/teorth/equational_theories) project.
- [ ] depends on: #25966
- [ ] depends on: #27672
- [ ] depends on: #27673
- [ ] depends on: #27678
---
[](https://gitpod.io/from-referrer/)
|
t-group-theory
merge-conflict
blocked-by-other-PR
|
364/0 |
Mathlib.lean,Mathlib/GroupTheory/FreeGroup/Basic.lean,Mathlib/GroupTheory/FreeGroup/CyclicallyReduced.lean,Mathlib/GroupTheory/FreeGroup/Reduce.lean |
4 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
30-65362 30 days ago |
30-65363 30 days ago |
0-2410 40 minutes |
27290 |
themathqueen author:themathqueen |
feat: `Star`, `StarAddMonoid`, and `StarModule` instances for tensor products |
This pr defines the `Star`, `StarAddMonoid` and `StarModule` instances on tensor product spaces.
---
- [ ] depends on: #27288
[](https://gitpod.io/from-referrer/)
|
t-algebra
blocked-by-other-PR
label:t-algebra$ |
85/27 |
Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/ChangeOfRings.lean,Mathlib/LinearAlgebra/TensorProduct/Basic.lean,Mathlib/LinearAlgebra/TensorProduct/Star.lean,Mathlib/RingTheory/Coalgebra/Hom.lean |
5 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
30-48159 30 days ago |
55-78078 1 month ago |
0-840 14 minutes |
27897 |
grunweg author:grunweg |
feat: check indentation of doc-strings |
Likely will require further adaptations to mathlib. May land piece-wise. But at first, let's see how big the overall fallout actually is.
(So far: 100 lines of implementation and tests, and 170 lines of fix-ups; which are probably mostly complete, but not entirely.)
---
- [ ] depends on: #27898
[](https://gitpod.io/from-referrer/)
|
t-linter
awaiting-CI
merge-conflict
blocked-by-other-PR
|
339/20 |
Mathlib/Algebra/Order/Hom/Basic.lean,Mathlib/Algebra/Polynomial/EraseLead.lean,Mathlib/Algebra/Polynomial/Inductions.lean,Mathlib/Algebra/Polynomial/Laurent.lean,Mathlib/CategoryTheory/Bicategory/NaturalTransformation/Oplax.lean,Mathlib/CategoryTheory/ConcreteCategory/Basic.lean,Mathlib/CategoryTheory/Enriched/Opposite.lean,Mathlib/CategoryTheory/Filtered/Basic.lean,Mathlib/CategoryTheory/Monoidal/Category.lean,Mathlib/CategoryTheory/Monoidal/Functor.lean,Mathlib/CategoryTheory/Monoidal/Limits.lean,Mathlib/CategoryTheory/NatIso.lean,Mathlib/Combinatorics/Configuration.lean,Mathlib/Data/Fin/Basic.lean,Mathlib/Data/Finsupp/MonomialOrder.lean,Mathlib/Data/Finsupp/MonomialOrder/DegLex.lean,Mathlib/Data/List/EditDistance/Defs.lean,Mathlib/Data/PNat/Xgcd.lean,Mathlib/Data/Part.lean,Mathlib/Geometry/Manifold/LocalDiffeomorph.lean,Mathlib/GroupTheory/GroupAction/MultiplePrimitivity.lean,Mathlib/MeasureTheory/Function/AEEqOfIntegral.lean,Mathlib/NumberTheory/RamificationInertia/Basic.lean,Mathlib/Order/Filter/Partial.lean,Mathlib/Order/Interval/Finset/Defs.lean,Mathlib/RingTheory/DividedPowers/Basic.lean,Mathlib/Tactic/ComputeDegree.lean,Mathlib/Tactic/FunProp/Decl.lean,Mathlib/Tactic/FunProp/Theorems.lean,Mathlib/Tactic/FunProp/Types.lean,Mathlib/Tactic/Linter/DocString.lean,Mathlib/Tactic/MinImports.lean,Mathlib/Tactic/MoveAdd.lean,Mathlib/Tactic/RewriteSearch.lean,Mathlib/Tactic/ToAdditive/Frontend.lean,MathlibTest/DocString.lean,MathlibTest/slow_simp.lean |
37 |
5 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
30-15955 30 days ago |
30-15956 30 days ago |
0-1 1 second |
27996 |
grunweg author:grunweg |
feat: check indentation in doc-strings, medium version |
---
- [ ] depends on: #27898
[](https://gitpod.io/from-referrer/)
|
merge-conflict
blocked-by-other-PR
WIP
|
816/505 |
Mathlib/Algebra/Algebra/Spectrum/Basic.lean,Mathlib/Algebra/ContinuedFractions/Basic.lean,Mathlib/Algebra/EuclideanDomain/Defs.lean,Mathlib/Algebra/Field/Subfield/Basic.lean,Mathlib/Algebra/Group/Subgroup/Finite.lean,Mathlib/Algebra/Lie/Classical.lean,Mathlib/Algebra/Lie/OfAssociative.lean,Mathlib/Algebra/Module/LinearMap/Polynomial.lean,Mathlib/Algebra/MvPolynomial/Equiv.lean,Mathlib/Algebra/Order/Antidiag/Prod.lean,Mathlib/Algebra/Order/Hom/Basic.lean,Mathlib/Algebra/Polynomial/EraseLead.lean,Mathlib/Algebra/Polynomial/Inductions.lean,Mathlib/Algebra/Polynomial/Laurent.lean,Mathlib/CategoryTheory/Abelian/Basic.lean,Mathlib/CategoryTheory/Adjunction/AdjointFunctorTheorems.lean,Mathlib/CategoryTheory/Bicategory/NaturalTransformation/Oplax.lean,Mathlib/CategoryTheory/Comma/Arrow.lean,Mathlib/CategoryTheory/Comma/Over/Basic.lean,Mathlib/CategoryTheory/ConcreteCategory/Basic.lean,Mathlib/CategoryTheory/Enriched/Opposite.lean,Mathlib/CategoryTheory/EpiMono.lean,Mathlib/CategoryTheory/Equivalence.lean,Mathlib/CategoryTheory/EssentialImage.lean,Mathlib/CategoryTheory/Filtered/Basic.lean,Mathlib/CategoryTheory/Generator/Basic.lean,Mathlib/CategoryTheory/Limits/ConeCategory.lean,Mathlib/CategoryTheory/Limits/Filtered.lean,Mathlib/CategoryTheory/Limits/FullSubcategory.lean,Mathlib/CategoryTheory/Limits/HasLimits.lean,Mathlib/CategoryTheory/Limits/Over.lean,Mathlib/CategoryTheory/Limits/Shapes/IsTerminal.lean,Mathlib/CategoryTheory/Limits/Shapes/WideEqualizers.lean,Mathlib/CategoryTheory/Limits/Types/Yoneda.lean,Mathlib/CategoryTheory/Monoidal/Category.lean,Mathlib/CategoryTheory/Monoidal/Functor.lean,Mathlib/CategoryTheory/Monoidal/Limits.lean,Mathlib/CategoryTheory/NatIso.lean,Mathlib/CategoryTheory/ObjectProperty/FullSubcategory.lean,Mathlib/CategoryTheory/Sites/Grothendieck.lean,Mathlib/CategoryTheory/Sites/Pretopology.lean,Mathlib/CategoryTheory/Sites/Sheaf.lean,Mathlib/CategoryTheory/Sites/Sieves.lean,Mathlib/CategoryTheory/Subobject/Comma.lean,Mathlib/CategoryTheory/Thin.lean,Mathlib/CategoryTheory/Yoneda.lean,Mathlib/Combinatorics/Configuration.lean,Mathlib/Combinatorics/Quiver/Symmetric.lean,Mathlib/Condensed/Equivalence.lean,Mathlib/Data/Bracket.lean,Mathlib/Data/Fin/Basic.lean,Mathlib/Data/Finset/NatAntidiagonal.lean,Mathlib/Data/Finsupp/MonomialOrder.lean,Mathlib/Data/Finsupp/MonomialOrder/DegLex.lean,Mathlib/Data/List/Defs.lean,Mathlib/Data/List/EditDistance/Defs.lean,Mathlib/Data/List/Rotate.lean,Mathlib/Data/Matrix/Composition.lean,Mathlib/Data/Multiset/Antidiagonal.lean,Mathlib/Data/Multiset/NatAntidiagonal.lean,Mathlib/Data/Num/Basic.lean,Mathlib/Data/Num/Bitwise.lean,Mathlib/Data/Ordmap/Ordnode.lean,Mathlib/Data/PNat/Xgcd.lean,Mathlib/Data/Part.lean,Mathlib/Data/Vector/Basic.lean,Mathlib/Data/Vector/Defs.lean,Mathlib/Geometry/Manifold/LocalDiffeomorph.lean,Mathlib/Geometry/RingedSpace/PresheafedSpace/Gluing.lean,Mathlib/GroupTheory/GroupAction/MultiplePrimitivity.lean,Mathlib/GroupTheory/GroupAction/Quotient.lean,Mathlib/LinearAlgebra/Finsupp/LinearCombination.lean,Mathlib/LinearAlgebra/InvariantBasisNumber.lean,Mathlib/LinearAlgebra/LinearIndependent/Basic.lean,Mathlib/MeasureTheory/Function/AEEqOfIntegral.lean,Mathlib/MeasureTheory/Group/Action.lean,Mathlib/NumberTheory/FLT/Basic.lean,Mathlib/NumberTheory/RamificationInertia/Basic.lean,Mathlib/Order/Filter/Partial.lean,Mathlib/Order/Interval/Finset/Defs.lean,Mathlib/RingTheory/DividedPowers/Basic.lean,Mathlib/RingTheory/Ideal/Maximal.lean,Mathlib/RingTheory/Ideal/Operations.lean,Mathlib/RingTheory/Ideal/Prod.lean,Mathlib/RingTheory/Ideal/Quotient/Basic.lean,Mathlib/RingTheory/Ideal/Quotient/Operations.lean,Mathlib/RingTheory/Localization/Defs.lean,Mathlib/SetTheory/Cardinal/Cofinality.lean,Mathlib/SetTheory/Ordinal/Family.lean,Mathlib/SetTheory/Ordinal/FixedPoint.lean,Mathlib/Tactic/Algebraize.lean,Mathlib/Tactic/Bound/Attribute.lean,Mathlib/Tactic/ComputeDegree.lean,Mathlib/Tactic/FunProp/Decl.lean,Mathlib/Tactic/FunProp/Theorems.lean,Mathlib/Tactic/FunProp/Types.lean,Mathlib/Tactic/Linter/DocString.lean,Mathlib/Tactic/MinImports.lean,Mathlib/Tactic/MoveAdd.lean,Mathlib/Tactic/RewriteSearch.lean |
107 |
6 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
30-15830 30 days ago |
30-15831 30 days ago |
0-1 1 second |
27980 |
smmercuri author:smmercuri |
feat: dimensions of completions at infinite place extensions |
This PR continues the work from #24853.
Original PR: https://github.com/leanprover-community/mathlib4/pull/24853
---
- [ ] depends on: #27977
- [ ] depends on: #27978
- [ ] depends on: #27979
- [ ] depends on: #27974
- [ ] depends on: #27975
- [ ] depends on: #27976 |
large-import
t-number-theory
merge-conflict
blocked-by-other-PR
|
878/1 |
Mathlib.lean,Mathlib/Analysis/Normed/Field/WithAbs.lean,Mathlib/NumberTheory/NumberField/InfinitePlace/Basic.lean,Mathlib/NumberTheory/NumberField/InfinitePlace/Dimension.lean,Mathlib/NumberTheory/NumberField/InfinitePlace/Embeddings.lean,Mathlib/NumberTheory/NumberField/InfinitePlace/Ramification.lean |
6 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
29-63924 29 days ago |
29-63924 29 days ago |
0-3752 1 hour |
7873 |
astrainfinita author:astrainfinita |
perf: reorder `extends` and change instance priority in algebra hierarchy |
There are no strict rules, but in general `Cancel` is dropped first, then `Comm`, then `Neg / Inv`, then `Assoc`. Not sure if there's a better way.
---
- [ ] depends on: #14712
- [x] depends on: #16638
- [ ] depends on: #18464
- [ ] depends on: #18468
- [ ] depends on: #18470
- [ ] depends on: #18472
- [ ] depends on: #18474
[](https://gitpod.io/from-referrer/)
|
slow-typeclass-synthesis
t-algebra
merge-conflict
blocked-by-other-PR
label:t-algebra$ |
494/204 |
Archive/Imo/Imo1998Q2.lean,Mathlib/Algebra/Algebra/Hom.lean,Mathlib/Algebra/Associated.lean,Mathlib/Algebra/BigOperators/Ring/List.lean,Mathlib/Algebra/Category/ModuleCat/Presheaf/Limits.lean,Mathlib/Algebra/DirectSum/Algebra.lean,Mathlib/Algebra/DirectSum/Internal.lean,Mathlib/Algebra/EuclideanDomain/Defs.lean,Mathlib/Algebra/EuclideanDomain/Field.lean,Mathlib/Algebra/Field/Basic.lean,Mathlib/Algebra/Field/Defs.lean,Mathlib/Algebra/Field/IsField.lean,Mathlib/Algebra/GCDMonoid/Basic.lean,Mathlib/Algebra/Group/Defs.lean,Mathlib/Algebra/Group/Ext.lean,Mathlib/Algebra/Group/InjSurj.lean,Mathlib/Algebra/Group/Opposite.lean,Mathlib/Algebra/Group/Prod.lean,Mathlib/Algebra/GroupWithZero/Basic.lean,Mathlib/Algebra/GroupWithZero/Defs.lean,Mathlib/Algebra/GroupWithZero/InjSurj.lean,Mathlib/Algebra/GroupWithZero/Prod.lean,Mathlib/Algebra/GroupWithZero/Semiconj.lean,Mathlib/Algebra/GroupWithZero/Units/Basic.lean,Mathlib/Algebra/Homology/Embedding/Basic.lean,Mathlib/Algebra/Homology/HomotopyCategory/DegreewiseSplit.lean,Mathlib/Algebra/Homology/HomotopyCategory/ShiftSequence.lean,Mathlib/Algebra/Lie/Basic.lean,Mathlib/Algebra/MonoidAlgebra/Grading.lean,Mathlib/Algebra/Order/AddGroupWithTop.lean,Mathlib/Algebra/Order/Field/Canonical/Defs.lean,Mathlib/Algebra/Order/Field/Defs.lean,Mathlib/Algebra/Order/Group/Abs.lean,Mathlib/Algebra/Order/Group/Defs.lean,Mathlib/Algebra/Order/GroupWithZero/Canonical.lean,Mathlib/Algebra/Order/Kleene.lean,Mathlib/Algebra/Order/Monoid/Defs.lean,Mathlib/Algebra/Order/Ring/Canonical.lean,Mathlib/Algebra/Order/Ring/Defs.lean,Mathlib/Algebra/Polynomial/Roots.lean,Mathlib/Algebra/Quaternion.lean,Mathlib/Algebra/Ring/BooleanRing.lean,Mathlib/Algebra/Ring/Defs.lean,Mathlib/Algebra/Ring/Ext.lean,Mathlib/Algebra/Ring/InjSurj.lean,Mathlib/Algebra/Ring/Rat.lean,Mathlib/Algebra/Tropical/Basic.lean,Mathlib/Analysis/Fourier/FourierTransformDeriv.lean,Mathlib/Analysis/InnerProductSpace/Orientation.lean,Mathlib/Analysis/InnerProductSpace/Symmetric.lean,Mathlib/Analysis/Normed/Field/Basic.lean,Mathlib/Analysis/Normed/Group/Basic.lean,Mathlib/Analysis/NormedSpace/Star/Multiplier.lean,Mathlib/CategoryTheory/Preadditive/FunctorCategory.lean,Mathlib/CategoryTheory/Preadditive/SingleObj.lean,Mathlib/CategoryTheory/Triangulated/Functor.lean,Mathlib/Data/Finset/NoncommProd.lean,Mathlib/Data/Int/Cast/Defs.lean,Mathlib/Data/Nat/Cast/Defs.lean,Mathlib/Data/Nat/Choose/Multinomial.lean,Mathlib/Data/Num/Lemmas.lean,Mathlib/Data/Rat/Denumerable.lean,Mathlib/Data/Real/ENatENNReal.lean,Mathlib/Dynamics/Ergodic/AddCircle.lean,Mathlib/FieldTheory/KummerExtension.lean,Mathlib/GroupTheory/Congruence/Basic.lean,Mathlib/GroupTheory/MonoidLocalization.lean,Mathlib/GroupTheory/SpecificGroups/Alternating.lean,Mathlib/GroupTheory/Torsion.lean,Mathlib/Init/ZeroOne.lean,Mathlib/LinearAlgebra/LinearPMap.lean,Mathlib/LinearAlgebra/Orientation.lean,Mathlib/LinearAlgebra/QuadraticForm/Basic.lean,Mathlib/LinearAlgebra/TensorPower.lean,Mathlib/LinearAlgebra/TensorProduct/Basic.lean,Mathlib/LinearAlgebra/TensorProduct/Graded/External.lean,Mathlib/MeasureTheory/Decomposition/Jordan.lean,Mathlib/MeasureTheory/Decomposition/SignedLebesgue.lean,Mathlib/NumberTheory/ArithmeticFunction.lean,Mathlib/NumberTheory/LegendreSymbol/GaussEisensteinLemmas.lean,Mathlib/NumberTheory/RamificationInertia.lean,Mathlib/NumberTheory/WellApproximable.lean,Mathlib/NumberTheory/Zsqrtd/QuadraticReciprocity.lean,Mathlib/Order/Filter/Germ.lean,Mathlib/Order/Interval/Finset/Box.lean,Mathlib/RingTheory/Bialgebra/Hom.lean,Mathlib/RingTheory/Coalgebra/Hom.lean,Mathlib/RingTheory/DiscreteValuationRing/Basic.lean,Mathlib/RingTheory/Filtration.lean,Mathlib/RingTheory/Henselian.lean,Mathlib/RingTheory/Ideal/IsPrincipal.lean,Mathlib/RingTheory/Ideal/LocalRing.lean,Mathlib/RingTheory/Ideal/Norm.lean,Mathlib/RingTheory/Localization/Integral.lean,Mathlib/RingTheory/MvPolynomial/Symmetric.lean,Mathlib/RingTheory/TensorProduct/Basic.lean,Mathlib/RingTheory/TensorProduct/MvPolynomial.lean,Mathlib/RingTheory/UniqueFactorizationDomain.lean,Mathlib/RingTheory/Valuation/ValuationSubring.lean,Mathlib/Tactic/Positivity/Core.lean |
104 |
84 |
['MichaelStollBayreuth', 'astrainfinita', 'github-actions', 'kim-em', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'mattrobball'] |
nobody |
28-63810 28 days ago |
424-35363 1 year ago |
7-77799 7 days |
26985 |
agjftucker author:agjftucker |
feat(Analysis/Calculus/Implicit): define implicitFunOfBivariate |
This PR continues the work from #16743.
Original PR: https://github.com/leanprover-community/mathlib4/pull/16743
---
- [ ] depends on: #26300
[](https://gitpod.io/from-referrer/) |
large-import
new-contributor
t-analysis
blocked-by-other-PR
|
282/9 |
Mathlib.lean,Mathlib/Analysis/Calculus/FDeriv/Partial.lean,Mathlib/Analysis/Calculus/Implicit.lean,Mathlib/Analysis/Normed/Module/Convex.lean,Mathlib/Order/Filter/Prod.lean |
5 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
28-35454 28 days ago |
31-67303 1 month ago |
0-213 3 minutes |
28530 |
nonisomorphiclinearmap author:nonisomorphiclinearmap |
feat(Combinatorics/SimplicialComplex/Topology): add standard simplices and geometric realisation (colimit + functoriality) |
Introduce the standard simplex on a finite vertex set and build the geometric realisation |X| of a simplicial complex. Prove that |X| is the colimit of the face diagram δ_X : X.faces ⥤ TopCat, and define the induced map on realisations |φ| : |X| ⟶ |Y| for a simplicial map φ. Show that the abstract map from colimit functoriality agrees with the concrete push-forward of barycentric coordinates. Package these into a functor SimplicialComplexCat ⥤ TopCat.
---
This is our first contribution to mathlib. This work was done as part of the Fields Institute Summer Undergraduate Program on formalization in topological combinatorics. Eventually, we aim to formalize Lovasz's proof of the Kneser Conjecture and this lays the groundwork to do this.
We would like to acknowledge the Fields Institute for Research in Mathematical Sciences for their sponsorship. We would also like to thank our supervisors, Professor Chris Kapulkin and Mr. Daniel Carranza, for their guidance and support throughout this project. I would also like to thank our group members Sebastian Kumar, Tom Lindquist and Quang Minh Nguyen for our fruitful discussions.
- [ ] depends on: #28125 |
new-contributor
t-combinatorics
blocked-by-other-PR
|
1826/0 |
Mathlib.lean,Mathlib/Combinatorics/SimplicialComplex/Basic.lean,Mathlib/Combinatorics/SimplicialComplex/Category.lean,Mathlib/Combinatorics/SimplicialComplex/FacePoset.lean,Mathlib/Combinatorics/SimplicialComplex/Hom.lean,Mathlib/Combinatorics/SimplicialComplex/Topology/GeomReal/Basic.lean,Mathlib/Combinatorics/SimplicialComplex/Topology/GeomReal/Colimit.lean,Mathlib/Combinatorics/SimplicialComplex/Topology/GeomReal/Diagram.lean,Mathlib/Combinatorics/SimplicialComplex/Topology/GeomReal/Functor.lean,Mathlib/Combinatorics/SimplicialComplex/Topology/GeomReal/Map.lean,Mathlib/Combinatorics/SimplicialComplex/Topology/Simplex.lean,Mathlib/Combinatorics/SimplicialComplex/Topology/SimplexMap.lean |
12 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
27-43570 27 days ago |
27-50147 27 days ago |
0-591 9 minutes |
27821 |
BGuillemet author:BGuillemet |
feat(CategoryTheory/Sites/Sheaf): functorial version of Sheaf.homEquiv |
Add two functorial versions of Sheaf.homEquiv, one using `yoneda` and the other using `coyoneda`.
---
- [ ] depends on: #27819
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-category-theory
merge-conflict
blocked-by-other-PR
|
182/37 |
Mathlib/CategoryTheory/Sites/Sheaf.lean,Mathlib/CategoryTheory/Yoneda.lean |
2 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
25-83553 25 days ago |
25-83554 25 days ago |
0-2066 34 minutes |
27557 |
chrisflav author:chrisflav |
feat(RingTheory/KrullDimension): dimension of `R / (x)` for a nonzerodivisor |
We show that if `R` is Noetherian and `x` is a nonzerodivisor contained in the Jacobson radical of `R`, then `dim R / (x) + 1 = dim R`.
---
- [ ] depends on: #27538
- [ ] depends on: #27510
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
large-import
merge-conflict
blocked-by-other-PR
|
509/1 |
Mathlib/Algebra/Module/SpanRank.lean,Mathlib/Data/Finset/Card.lean,Mathlib/Data/Fintype/Card.lean,Mathlib/Logic/Function/Basic.lean,Mathlib/Order/KrullDimension.lean,Mathlib/RingTheory/Ideal/GoingDown.lean,Mathlib/RingTheory/Ideal/Height.lean,Mathlib/RingTheory/Ideal/KrullsHeightTheorem.lean,Mathlib/RingTheory/Ideal/Maps.lean,Mathlib/RingTheory/Ideal/MinimalPrime/Basic.lean,Mathlib/RingTheory/Ideal/Over.lean,Mathlib/RingTheory/Ideal/Quotient/Operations.lean,Mathlib/RingTheory/KrullDimension/Basic.lean,Mathlib/RingTheory/KrullDimension/NonZeroDivisors.lean,Mathlib/RingTheory/KrullDimension/PID.lean,Mathlib/RingTheory/Localization/AtPrime.lean,Mathlib/RingTheory/Spectrum/Prime/RingHom.lean |
17 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
25-83287 25 days ago |
39-61420 1 month ago |
0-562 9 minutes |
27542 |
chrisflav author:chrisflav |
feat(RingTheory/KrullDimension): dimension of polynomial ring |
We show that for a Noetherian ring `R`, `dim R[X] = dim R + 1`.
Co-authored by: Sihan Su
Co-authored by: Yi Song
---
- [ ] depends on: #27520
- [ ] depends on: #27538
- [ ] depends on: #27510
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
large-import
merge-conflict
blocked-by-other-PR
|
474/3 |
Mathlib/Algebra/Module/SpanRank.lean,Mathlib/Data/Finset/Card.lean,Mathlib/Data/Fintype/Card.lean,Mathlib/Logic/Function/Basic.lean,Mathlib/Order/KrullDimension.lean,Mathlib/RingTheory/Ideal/GoingDown.lean,Mathlib/RingTheory/Ideal/Height.lean,Mathlib/RingTheory/Ideal/KrullsHeightTheorem.lean,Mathlib/RingTheory/Ideal/Maps.lean,Mathlib/RingTheory/Ideal/MinimalPrime/Basic.lean,Mathlib/RingTheory/Ideal/Over.lean,Mathlib/RingTheory/Ideal/Quotient/Operations.lean,Mathlib/RingTheory/KrullDimension/Basic.lean,Mathlib/RingTheory/KrullDimension/PID.lean,Mathlib/RingTheory/KrullDimension/Polynomial.lean,Mathlib/RingTheory/Localization/AtPrime/Basic.lean,Mathlib/RingTheory/Spectrum/Prime/RingHom.lean |
17 |
n/a |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
25-83286 25 days ago |
unknown |
unknown |
27979 |
smmercuri author:smmercuri |
feat: `RamifiedExtension` and `UnramifiedExtension` types for `InfinitePlace.Extension`s |
This PR continues the work from #24882.
Original PR: https://github.com/leanprover-community/mathlib4/pull/24882
---
- [ ] depends on: #27977 |
t-number-theory
blocked-by-other-PR
|
242/0 |
Mathlib/NumberTheory/NumberField/InfinitePlace/Embeddings.lean,Mathlib/NumberTheory/NumberField/InfinitePlace/Ramification.lean |
2 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
riccardobrasca assignee:riccardobrasca |
25-79977 25 days ago |
38-85190 1 month ago |
0-278 4 minutes |
28502 |
gilesgshaw author:gilesgshaw |
feat(Logic/Basic): avoid unnecessary uses of choice |
Certain proofs are modified to remove a dependence on the axoim of choice
---
- [ ] depends on: #28623
|
new-contributor
t-logic
merge-conflict
awaiting-author
blocked-by-other-PR
|
83/74 |
Mathlib/Logic/Basic.lean |
1 |
7 |
['Ruben-VandeVelde', 'eric-wieser', 'gilesgshaw', 'github-actions', 'kim-em', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
25-18613 25 days ago |
25-18614 25 days ago |
0-35689 9 hours |
26831 |
AntoineChambert-Loir author:AntoineChambert-Loir |
feat(GroupTheory/SpecificGroups/Alternating/MaximalSubgroups): maximal subgroups of the alternating group |
This proves the first case (intransitive) of the O'Nan-Scott classification of maximal subgroups of the alternating group.
---
- [ ] depends on: #26457
- [ ] depends on: #26282
- [x] depends on: #26281
- [x] depends on: #26280
- [x] depends on: #26279
[](https://gitpod.io/from-referrer/)
|
t-group-theory
large-import
blocked-by-other-PR
|
2169/145 |
Mathlib.lean,Mathlib/Data/Set/Card.lean,Mathlib/GroupTheory/GroupAction/Jordan.lean,Mathlib/GroupTheory/GroupAction/MultiplePrimitivity.lean,Mathlib/GroupTheory/GroupAction/MultipleTransitivity.lean,Mathlib/GroupTheory/GroupAction/Primitive.lean,Mathlib/GroupTheory/GroupAction/SubMulAction/OfFixingSubgroup.lean,Mathlib/GroupTheory/GroupAction/SubMulAction/OfStabilizer.lean,Mathlib/GroupTheory/Perm/Cycle/Basic.lean,Mathlib/GroupTheory/Perm/Cycle/Type.lean,Mathlib/GroupTheory/Perm/MaximalSubgroups.lean,Mathlib/GroupTheory/SpecificGroups/Alternating.lean,Mathlib/GroupTheory/SpecificGroups/Alternating/MaximalSubgroups.lean,Mathlib/SetTheory/Cardinal/Embedding.lean,docs/references.bib |
15 |
n/a |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
25-12102 25 days ago |
unknown |
unknown |
26315 |
EtienneC30 author:EtienneC30 |
feat: continuous sesquilinear forms |
Introduce an abbreviation `ContinuousSesquilinForm` for `E →L⋆[𝕜] E →L[𝕜] 𝕜`. This is needed in the Brownian motion project, as a Gaussian measure is represented by its mean and its covariance bilinear form, which is a positive semidefinite bilinear form.
---
- [x] depends on: #26274
- [ ] depends on: #28052
From Brownian motion
[](https://gitpod.io/from-referrer/)
|
t-analysis
merge-conflict
blocked-by-other-PR
|
469/39 |
Counterexamples/QuadraticForm.lean,Mathlib.lean,Mathlib/Algebra/Lie/TraceForm.lean,Mathlib/Analysis/NormedSpace/ContinuousSesquilinForm.lean,Mathlib/LinearAlgebra/BilinearForm/Properties.lean,Mathlib/LinearAlgebra/BilinearForm/TensorProduct.lean,Mathlib/LinearAlgebra/Matrix/BilinearForm.lean,Mathlib/LinearAlgebra/Matrix/Hermitian.lean,Mathlib/LinearAlgebra/QuadraticForm/Basic.lean,Mathlib/LinearAlgebra/QuadraticForm/Dual.lean,Mathlib/LinearAlgebra/RootSystem/Finite/CanonicalBilinear.lean,Mathlib/LinearAlgebra/RootSystem/OfBilinear.lean,Mathlib/LinearAlgebra/RootSystem/RootPositive.lean,Mathlib/LinearAlgebra/SesquilinearForm.lean,Mathlib/LinearAlgebra/SesquilinearForm/Basic.lean,Mathlib/LinearAlgebra/SesquilinearForm/IsPosSemidef.lean |
16 |
10 |
['EtienneC30', 'RemyDegenne', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
24-82195 24 days ago |
24-82196 24 days ago |
0-0 0 seconds |
27353 |
themathqueen author:themathqueen |
chore(LinearAlgebra/TensorProduct/Basic): semi-linearizing part 1 |
This continues the work from: #27310 (original PR: #24208).
The only extra definition is `LinearMap.compr₂ₛₗ` for the semi-linear version of `LinearMap.compr₂`.
Co-authored-by: @ADedecker
---
- [x] depends on: #27467
- [ ] depends on: #27288
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
blocked-by-other-PR
label:t-algebra$ |
230/187 |
Mathlib/Algebra/Category/ModuleCat/ChangeOfRings.lean,Mathlib/Algebra/Category/ModuleCat/Monoidal/Basic.lean,Mathlib/Algebra/Category/ModuleCat/Monoidal/Closed.lean,Mathlib/Algebra/Lie/TensorProduct.lean,Mathlib/CategoryTheory/Monoidal/Internal/Module.lean,Mathlib/LinearAlgebra/BilinearForm/TensorProduct.lean,Mathlib/LinearAlgebra/Coevaluation.lean,Mathlib/LinearAlgebra/Contraction.lean,Mathlib/LinearAlgebra/DirectSum/TensorProduct.lean,Mathlib/LinearAlgebra/Dual/Lemmas.lean,Mathlib/LinearAlgebra/TensorProduct/Basic.lean,Mathlib/LinearAlgebra/TensorProduct/Tower.lean,Mathlib/LinearAlgebra/Trace.lean,Mathlib/RepresentationTheory/Rep.lean,Mathlib/RingTheory/Coalgebra/Hom.lean |
15 |
15 |
['eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'themathqueen'] |
nobody |
24-19774 24 days ago |
24-19774 24 days ago |
2-62342 2 days |
27198 |
robin-carlier author:robin-carlier |
feat(CategoryTheory/Monoidal/DayConvolution): the Yoneda embedding is monoidal (for Day convolution) |
We show that the Yoneda embedding is monoidal when we interpret its target category as Day presheaves (i.e presheaves with the Day convolution monoidal structure). The actual way we prove it is by registering a `LawfulDayConvolutionMonoidalCategoryStruct Cᵒᵖ (Type v₁) C`, for which the "interpretation" functor `C ⥤ Cᵒᵖ ⥤ Type v₁` is the Yoneda embedding. This allows to state a result independently of any size constraint on `C`.
Then, we specialize to the case of a small category `C`, in this case, using the fact that the relevant colimit of preseaves exist, we use the fact that the interpretation functor induces a monoidal functor to put a `Monoidal` instance on the functor `dayYoneda : C ⥤ (Cᵒᵖ ⊛⥤ Type v₁) := yoneda ⋙ (equiv Cᵒᵖ _).inverse`.
---
I was unsure about which form of simp lemmas we want for characterization of the monoidal structure on `dayYoneda`. I opted for making the "fully applied" lemmas simp, but still leaves the "unapplied" ones as non-simp just in case.
- [ ] depends on: #27175
- [ ] depends on: #25732
[](https://gitpod.io/from-referrer/)
|
file-removed
t-category-theory
merge-conflict
blocked-by-other-PR
|
1847/26 |
Mathlib.lean,Mathlib/CategoryTheory/Functor/KanExtension/Basic.lean,Mathlib/CategoryTheory/Monoidal/DayConvolution.lean,Mathlib/CategoryTheory/Monoidal/DayConvolution/DayFunctor.lean,Mathlib/CategoryTheory/Monoidal/DayConvolution/Types.lean,Mathlib/CategoryTheory/Monoidal/Internal/Limits.lean,Mathlib/CategoryTheory/Monoidal/Limits/Basic.lean,Mathlib/CategoryTheory/Monoidal/Limits/Preserves.lean |
8 |
5 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
24-17146 24 days ago |
24-17146 24 days ago |
0-21 21 seconds |
23831 |
vasnesterov author:vasnesterov |
feat(Analysis): binomial series convergence |
Prove
* `one_add_cpow_hasFPowerSeriesOnBall_zero`: for complex `a` and `|x| < 1`, the binomial series converges to `(1 + x).cpow a`.
* `one_add_rpow_hasFPowerSeriesOnBall_zero`: the variant of the above for reals.
---
- [x] depends on: #27537
- [ ] depends on: #26267
- [x] depends on: #26268
[](https://gitpod.io/from-referrer/)
|
t-analysis
merge-conflict
blocked-by-other-PR
|
606/6 |
Mathlib.lean,Mathlib/Analysis/Analytic/Basic.lean,Mathlib/Analysis/Analytic/Binomial.lean,Mathlib/Analysis/Analytic/ChangeOrigin.lean,Mathlib/Analysis/Analytic/Constructions.lean,Mathlib/Analysis/Calculus/FormalMultilinearSeries.lean,Mathlib/Analysis/Calculus/IteratedDeriv/Defs.lean,Mathlib/Analysis/Calculus/IteratedDeriv/Lemmas.lean,Mathlib/Analysis/NormedSpace/Connected.lean,Mathlib/NumberTheory/NumberField/CanonicalEmbedding/Basic.lean,Mathlib/RingTheory/Binomial.lean,scripts/noshake.json |
12 |
2 |
['leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
24-3110 24 days ago |
157-71328 5 months ago |
0-822 13 minutes |
26719 |
AntoineChambert-Loir author:AntoineChambert-Loir |
feat(RingTheory/PolynomialLaw/Basic): extends polynomial laws to arbitrary universes |
The definition of polynomial laws restricts its operations to a fixed universe.
This PR constructs the extension to any universe.
This is part of the project of studying divided powers on rings, in particular, for studying
the universal divided power algebra of a module.
Co-authored-by: María-Inés de Frutos Fernández @mariainesdff
---
- [x] depends on: #26717
- [ ] depends on: #26277
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
large-import
blocked-by-other-PR
|
969/7 |
Mathlib.lean,Mathlib/Algebra/Ring/Subsemiring/Basic.lean,Mathlib/Algebra/RingQuot.lean,Mathlib/LinearAlgebra/TensorProduct/Tower.lean,Mathlib/RingTheory/Congruence/Basic.lean,Mathlib/RingTheory/Congruence/Defs.lean,Mathlib/RingTheory/Congruence/Hom.lean,Mathlib/RingTheory/PolynomialLaw/Basic.lean |
8 |
4 |
['acmepjz', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
24-416 24 days ago |
39-4066 1 month ago |
0-1757 29 minutes |
28499 |
yoh-tanimoto author:yoh-tanimoto |
feat(MeasureTheory/VectorMeasure): add integral of a vector-valued function against a vector measure |
add `VectorMeasureWithPairing.integral` for normed vector spaces `E`, `F`, a Banach space `G` , a continuous linear pairing `B : E →L[ℝ] F →L[ℝ] → G` and an `F`-valued vector measure `μ`, which should be informally written as `∫ B (f x) ∂μ x`.
motivation: there are natural vector measures such as signed measures and complex measures, and their integrals appear naturally e.g. in a proof of the spectral theorem for general bounded normal operators on a Hilbert space.
- [ ] depends on: #26160 for the definition and lemmas about the total variation of a vector measure. |
t-measure-probability
blocked-by-other-PR
|
651/0 |
Mathlib.lean,Mathlib/MeasureTheory/VectorMeasure/Integral.lean,Mathlib/MeasureTheory/VectorMeasure/Variation/Defs.lean,Mathlib/MeasureTheory/VectorMeasure/Variation/Lemmas.lean |
4 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
23-78527 23 days ago |
28-39344 28 days ago |
0-3692 1 hour |
25906 |
pfaffelh author:pfaffelh |
feat (Topology/Compactness/CompactSystem): Closed and compact square cylinders form a compact system. |
feat (Topology/Compactness/CompactSystem): Closed and compact square cylinders form a
compact system.
A square cylinder is a set of the form `s.pi t` in a product space. A closed compact square cylinder has `IsClosed (t i)` and `IsCompact (t i)` for all `i ∈ s`. This set system is a compact system (as introduced in PR #25899).
Streamline the definition of square cylinders in MeasureTheory/Constructions/Cylinders on the way.
Co-authors: Rémy Degenne remy.degenne@inria.fr
---
- [ ] depends on: #25899
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #24542.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/24542* |
t-topology
blocked-by-other-PR
|
716/65 |
Mathlib.lean,Mathlib/Data/Set/Accumulate.lean,Mathlib/Data/Set/Dissipate.lean,Mathlib/Data/Set/Prod.lean,Mathlib/MeasureTheory/Constructions/Cylinders.lean,Mathlib/MeasureTheory/Constructions/ProjectiveFamilyContent.lean,Mathlib/MeasureTheory/PiSystem.lean,Mathlib/Topology/Compactness/CompactSystem.lean |
8 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
23-4952 23 days ago |
23-46536 23 days ago |
0-383 6 minutes |
25900 |
pfaffelh author:pfaffelh |
feat (Topology/Compactness/CompactSystem): Set system of finite unions of sets in a compact system is again a compact system |
feat (Topology/Compactness/CompactSystem): The set system of finite unions of sets in a compact system is a compact system
A compact system is a set system with the following property: If all finite intersections of a sequence in the set system is non-empty, the countable intersection is not empty.
Starting with a compact system, consider the finite unions of sets in the copact system. Such sets again form a compact system (`IsCompactSystem.union.isCompactSystem`).
---
- [x] depends on: #24906
- [ ] depends on: #25899
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #24543.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/24543* |
t-topology
blocked-by-other-PR
|
996/66 |
Mathlib.lean,Mathlib/Data/Set/Accumulate.lean,Mathlib/Data/Set/Dissipate.lean,Mathlib/Data/Set/Prod.lean,Mathlib/MeasureTheory/Constructions/Cylinders.lean,Mathlib/MeasureTheory/Constructions/ProjectiveFamilyContent.lean,Mathlib/MeasureTheory/PiSystem.lean,Mathlib/Topology/Compactness/CompactSystem.lean |
8 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
22-78521 22 days ago |
22-78541 22 days ago |
0-850 14 minutes |
18805 |
astrainfinita author:astrainfinita |
refactor: deprecate `SemilinearMapClass` |
---
I'm not sure if we want to do this, but let's see if we can get a speed up from it first.
- [ ] depends on: #18755
- [ ] depends on: #18756
- [ ] depends on: #18806
[](https://gitpod.io/from-referrer/)
|
awaiting-bench
t-algebra
merge-conflict
blocked-by-other-PR
WIP
label:t-algebra$ |
546/318 |
Mathlib/Algebra/Algebra/Hom.lean,Mathlib/Algebra/Algebra/NonUnitalHom.lean,Mathlib/Algebra/Algebra/Rat.lean,Mathlib/Algebra/BigOperators/Balance.lean,Mathlib/Algebra/BigOperators/Expect.lean,Mathlib/Algebra/Category/ModuleCat/Basic.lean,Mathlib/Algebra/Group/Equiv/Basic.lean,Mathlib/Algebra/Group/Units/Equiv.lean,Mathlib/Algebra/GroupWithZero/Hom.lean,Mathlib/Algebra/Module/Equiv/Defs.lean,Mathlib/Algebra/Module/LinearMap/Defs.lean,Mathlib/Algebra/Module/LinearMap/Rat.lean,Mathlib/Algebra/Module/LocalizedModule/Int.lean,Mathlib/Algebra/Module/Submodule/EqLocus.lean,Mathlib/Algebra/Module/Submodule/Equiv.lean,Mathlib/Algebra/Module/Submodule/Ker.lean,Mathlib/Algebra/Module/Submodule/Map.lean,Mathlib/Algebra/Module/Submodule/Range.lean,Mathlib/Algebra/MvPolynomial/Equiv.lean,Mathlib/Algebra/Order/Hom/Monoid.lean,Mathlib/Algebra/Polynomial/AlgebraMap.lean,Mathlib/Algebra/Prime/Lemmas.lean,Mathlib/Algebra/Ring/Divisibility/Basic.lean,Mathlib/Algebra/Ring/Equiv.lean,Mathlib/Analysis/CStarAlgebra/Spectrum.lean,Mathlib/Analysis/LocallyConvex/WeakOperatorTopology.lean,Mathlib/Analysis/Normed/Algebra/Spectrum.lean,Mathlib/Analysis/Normed/Group/Uniform.lean,Mathlib/Analysis/Normed/Operator/LinearIsometry.lean,Mathlib/CategoryTheory/Limits/ConcreteCategory/WithAlgebraicStructures.lean,Mathlib/Combinatorics/Additive/FreimanHom.lean,Mathlib/Data/Complex/BigOperators.lean,Mathlib/FieldTheory/IsAlgClosed/AlgebraicClosure.lean,Mathlib/FieldTheory/SplittingField/Construction.lean,Mathlib/Geometry/Manifold/Instances/Sphere.lean,Mathlib/GroupTheory/GroupAction/Hom.lean,Mathlib/LinearAlgebra/Ray.lean,Mathlib/LinearAlgebra/Span.lean,Mathlib/RingTheory/Bialgebra/Equiv.lean,Mathlib/RingTheory/Flat/Basic.lean,Mathlib/RingTheory/HahnSeries/Addition.lean,Mathlib/RingTheory/Ideal/Norm.lean,Mathlib/RingTheory/Multiplicity.lean,Mathlib/RingTheory/Polynomial/Opposites.lean,Mathlib/RingTheory/RootsOfUnity/Basic.lean,Mathlib/Topology/Algebra/InfiniteSum/Basic.lean,Mathlib/Topology/Algebra/Module/Basic.lean,Mathlib/Topology/Algebra/Module/CharacterSpace.lean,Mathlib/Topology/Algebra/Module/FiniteDimension.lean,Mathlib/Topology/Algebra/Module/StrongTopology.lean,Mathlib/Topology/Algebra/Module/WeakDual.lean,Mathlib/Topology/Algebra/MulAction.lean,Mathlib/Topology/Homeomorph.lean,Mathlib/Topology/MetricSpace/Isometry.lean,scripts/no_lints_prime_decls.txt |
55 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
22-70448 22 days ago |
303-75117 9 months ago |
0-0 0 seconds |
25797 |
dagurtomas author:dagurtomas |
feat(Condensed): closed symmetric monoidal structure on light condensed modules |
---
- [ ] depends on: #25794
- [x] depends on: #24490
- [x] depends on: #24522
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #24523.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/24523* |
t-condensed
merge-conflict
blocked-by-other-PR
WIP
|
906/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/Monoidal/Braided/Transport.lean,Mathlib/CategoryTheory/Sites/Monoidal.lean,Mathlib/Condensed/Light/Monoidal.lean,Mathlib/Condensed/Light/Small.lean |
9 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
22-62746 22 days ago |
22-62747 22 days ago |
0-3 3 seconds |
19582 |
yu-yama author:yu-yama |
feat(GroupExtension/Abelian): define `OfMulDistribMulAction.equivH2` |
Mainly defines:
- `structure GroupExtension.OfMulDistribMulAction N G [MulDistribMulAction G N]`: group extensions of `G` by `N` where the multiplicative action of `G` on `N` is the conjugation
- `structure GroupExtension.OfMulDistribMulActionWithSection N G [MulDistribMulAction G N]`: group extensions with specific choices of sections
- `def GroupExtension.OfMulDistribMulAction.equivH2`: a bijection between the equivalence classes of group extensions and $H^2 (G, N)$
---
- [x] depends on: #20802 (split PR: contains changes to the `Defs` file)
- [x] depends on: #20998 (split PR: mainly adds the `Basic` file)
- [ ] depends on: #26670 (split PR: adds the first part of the `Abelian` file)
Here is a relevant TODO in Mathlib:
https://github.com/leanprover-community/mathlib4/blob/4e9fa40d7c480937e09cd6e47a591bd6f3b8be42/Mathlib/RepresentationTheory/GroupCohomology/LowDegree.lean#L46-L48
I would appreciate your comments.
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-algebra
merge-conflict
blocked-by-other-PR
label:t-algebra$ |
750/14 |
Mathlib.lean,Mathlib/GroupTheory/GroupExtension/Abelian.lean,Mathlib/GroupTheory/GroupExtension/Defs.lean,docs/references.bib |
4 |
5 |
['YaelDillies', 'erdOne', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
22-55121 22 days ago |
22-55122 22 days ago |
43-26015 43 days |
25903 |
pfaffelh author:pfaffelh |
feat(MeasureTheory): finite unions of sets in a semi-ring (in terms of measure theory) form a ring |
: Finite unions of sets in a semi-ring (in terms of measure theory) form a ring
The set containing finite unions of sets in a semi-ring are a ring.
Part of `MeasureTheory.SetSemiring` is moved to the new file `MeasureTheory.SetRing`.
---
- [ ] depends on: #25902 [contains changes in `SetSemiring` as well]
---
*This PR continues the work from #23117.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/23117* |
large-import
t-measure-probability
blocked-by-other-PR
|
648/131 |
Mathlib.lean,Mathlib/Algebra/Group/Pointwise/Finset/Basic.lean,Mathlib/Algebra/Module/Bimodule.lean,Mathlib/Data/Set/Lattice.lean,Mathlib/Data/Set/Pairwise/Lattice.lean,Mathlib/Data/Set/Prod.lean,Mathlib/MeasureTheory/MeasurableSpace/Pi.lean,Mathlib/MeasureTheory/Measure/AddContent.lean,Mathlib/MeasureTheory/PiSystem.lean,Mathlib/MeasureTheory/SetAlgebra.lean,Mathlib/MeasureTheory/SetRing.lean,Mathlib/MeasureTheory/SetSemiring.lean,Mathlib/Tactic.lean,Mathlib/Tactic/ExtractLets.lean,lake-manifest.json,lakefile.lean |
16 |
n/a |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
22-50898 22 days ago |
unknown |
unknown |
27215 |
kckennylau author:kckennylau |
feat(AlgebraicGeometry): Define the Zariski site on `CommRingCatᵒᵖ` |
We define the Zariski site on `CommRingCatᵒᵖ` by inducing the topology from `Scheme`, and then we show that this topology is equal to the one generated by the pretopology of finite, surjective, and standard open morphisms.
---
- [ ] depends on: #28614
- [x] depends on: #28615
[](https://gitpod.io/from-referrer/)
|
t-algebraic-geometry
blocked-by-other-PR
|
490/0 |
Mathlib.lean,Mathlib/AlgebraicGeometry/Sites/BigAffineZariski.lean,Mathlib/CategoryTheory/Sites/Finite.lean |
3 |
17 |
['chrisflav', 'github-actions', 'kckennylau', 'mathlib4-dependent-issues-bot'] |
chrisflav assignee:chrisflav |
21-66656 21 days ago |
25-45464 25 days ago |
0-42471 11 hours |
26871 |
grunweg author:grunweg |
feat: finite sum, difference, scalar product of differentiable sections is differentiable |
This mirrors the additions of #26674 to `mdifferentiable` sections.
Part of the path towards geodesics and the Levi-Civita connection.
Co-authored-by: Patrick Massot
---
TODO: make a follow-up PR adding analogues of the recent the `finsum` and `locallyFinite` results in `SmoothSection`.
- [ ] depends on: #26870 (and perhaps more/need to split afterwards)
[](https://gitpod.io/from-referrer/)
|
t-differential-geometry
merge-conflict
blocked-by-other-PR
|
470/3 |
Mathlib/Geometry/Manifold/VectorBundle/MDifferentiable.lean |
1 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
21-61162 21 days ago |
67-48726 2 months ago |
0-1058 17 minutes |
26466 |
robin-carlier author:robin-carlier |
feat(AlgebraicTopology/SimplexCategory/Augmented): the canonical monoid object in the augmented simplex category |
Show that in the augmented simplex category, `⦋0⦌` is an internal monoid object.
Future work will show that this is in fact the universal monoid object: for any monoidal category `C`, evaluation at `⦋0⦌` induces an equivalence of categories between `Mon_ C` and the category of monoidal functors from `AugmentedSimplexCategory` to `C`. The resulting augmented cosimplicial object one gets from this construction is sometimes called the "monoidal bar construction" attached to a monoid.
This PR was split from #25743.
---
- [ ] depends on: #25743
[](https://gitpod.io/from-referrer/)
|
t-algebraic-topology
t-category-theory
merge-conflict
blocked-by-other-PR
|
571/111 |
Mathlib.lean,Mathlib/AlgebraicTopology/SimplexCategory/Augmented.lean,Mathlib/AlgebraicTopology/SimplexCategory/Augmented/Basic.lean,Mathlib/AlgebraicTopology/SimplexCategory/Augmented/Mon_.lean,Mathlib/AlgebraicTopology/SimplexCategory/Augmented/Monoidal.lean,Mathlib/AlgebraicTopology/SimplexCategory/Basic.lean |
6 |
4 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
21-55836 21 days ago |
21-55837 21 days ago |
0-1708 28 minutes |
28246 |
Sebi-Kumar author:Sebi-Kumar |
feat(AlgebraicTopology/FundamentalGroupoid): the n-sphere is simply connected for n > 1 |
Prove that the `n`-dimensional sphere (i.e., the unit sphere centered at the origin in `(n + 1)`-dimensional real Euclidean space) is a simply connected space for `n > 1`. This proof follows Hatcher's "Algebraic Topology"; we first prove a general lemma about decomposing loops and then exploit the fact that non-surjective loops in the sphere are homotopically trivial.
Note: To get this file to build, I edited `Mathlib/Tactic/Linter/DirectoryDependency.lean` to remove the restrictions on AlgebraicTopology files importing Geometry, NumberTheory, and SetTheory files. Thank you to those who shared their expertise [here](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Warning.20that.20AlgebraicTopology.20can't.20import.20SetTheory/with/533833638). As I understand it, this is just a short-term solution, so I would appreciate feedback on what to do about this situation.
Note: I am unsure where exactly the file `SimplyConnectedSphere.lean` should go or whether that is an appropriate name for the file, so feedback there would be appreciated.
---
To provide additional context, this code was written as a part of the Fields Undergraduate Summer Research Program at the University of Western Ontario under the supervision of Chris Kapulkin and Daniel Carranza.
- [ ] depends on: #28208
- [ ] depends on: #28198
- [ ] depends on: #28185
- [ ] depends on: #28152
[](https://gitpod.io/from-referrer/)
|
t-algebraic-topology
new-contributor
blocked-by-other-PR
|
639/6 |
Mathlib.lean,Mathlib/AlgebraicTopology/FundamentalGroupoid/Basic.lean,Mathlib/AlgebraicTopology/FundamentalGroupoid/SimplyConnected.lean,Mathlib/AlgebraicTopology/FundamentalGroupoid/SimplyConnectedSphere.lean,Mathlib/Analysis/InnerProductSpace/PiL2.lean,Mathlib/Tactic/Linter/DirectoryDependency.lean,Mathlib/Topology/FoldTrans.lean,Mathlib/Topology/Path.lean,Mathlib/Topology/Subpath.lean |
9 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
21-53729 21 days ago |
32-50927 1 month ago |
0-23 23 seconds |
25488 |
VTrelat author:VTrelat |
feat(SetTheory/ZFC/Rationals): define rationals in ZFC |
Extend the model of ZFC with rationals: we define a proper type `ZFRat` representing integers based on pairs of `ZFInt` (enforcing the res to be nonzero) and following the usual construction of rationals.
---
[](https://gitpod.io/from-referrer/)
- [ ] depends on: #25483
- [ ] depends on: #25485
- [ ] depends on: #25486 |
t-set-theory
new-contributor
merge-conflict
blocked-by-other-PR
|
2070/0 |
Mathlib/Data/Set/Prod.lean,Mathlib/SetTheory/ZFC/Basic.lean,Mathlib/SetTheory/ZFC/Booleans.lean,Mathlib/SetTheory/ZFC/Integers.lean,Mathlib/SetTheory/ZFC/Rationals.lean |
5 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
21-19739 21 days ago |
21-19739 21 days ago |
0-1808 30 minutes |
28244 |
robin-carlier author:robin-carlier |
feat(CategoryTheory/Bicategory/NaturalTransformation): Icons |
We define icons (short for Identity Component Oplax Natural transformations) between lax functors in bicategories.
Such transformations bundle an oplax natural transformation, along with the assertion that the source and target functor agree on objects, and the fact that the app-component of the underlying natural transformation is the `eqToHom` morphism along that equality.
We define vertical composition of such natural transformations.
Strict associativity and strict unitality of the composition of icons will be the content of a follow-up PR.
In future work, icons will constitute the 2-cells of a strict bicategory structure on bicategories, with 1-cells (strictly unitary) pseudofunctors. This bicategory structure will define a category structure on strictly unitary pseudofunctors from `LocallyDiscrete (Fin n)` to a bicategory `C` (i.e "pseudo-composable arrows" in `C`), which will be part of the definition of the 2-nerve of `C`, which is a simplicial category that encodes higher compositions within a bicategory `C`.
---
- [ ] depends on: #25825
- [ ] depends on: #28243
[](https://gitpod.io/from-referrer/)
|
large-import
t-category-theory
awaiting-CI
blocked-by-other-PR
WIP
|
816/33 |
Mathlib.lean,Mathlib/CategoryTheory/Bicategory/EqToHom.lean,Mathlib/CategoryTheory/Bicategory/NaturalTransformation/Icon.lean,Mathlib/CategoryTheory/Bicategory/NaturalTransformation/Lax.lean,Mathlib/CategoryTheory/Bicategory/NaturalTransformation/Oplax.lean,Mathlib/CategoryTheory/Bicategory/Strict.lean,Mathlib/CategoryTheory/EqToHom.lean,scripts/noshake.json |
8 |
3 |
['github-actions', 'joelriou', 'mathlib4-dependent-issues-bot'] |
nobody |
21-875 21 days ago |
21-875 21 days ago |
0-1160 19 minutes |
28245 |
robin-carlier author:robin-carlier |
feat(CategoryTheory/Bicategory/NaturalTransformation/Icon): strict associativity and unitality of icon composition |
We show that the vertical composition of icons defined in #28244 satisfies strict associativity and strict unitality. This morally shows that icons are fit as the 2-cells of a bicategory structure on bicategories and lax functors, though we do not record an instance of this sort.
---
- [ ] depends on: #28244
[](https://gitpod.io/from-referrer/)
|
large-import
t-category-theory
awaiting-CI
blocked-by-other-PR
WIP
|
975/33 |
Mathlib.lean,Mathlib/CategoryTheory/Bicategory/EqToHom.lean,Mathlib/CategoryTheory/Bicategory/NaturalTransformation/Icon.lean,Mathlib/CategoryTheory/Bicategory/NaturalTransformation/Lax.lean,Mathlib/CategoryTheory/Bicategory/NaturalTransformation/Oplax.lean,Mathlib/CategoryTheory/Bicategory/Strict.lean,Mathlib/CategoryTheory/EqToHom.lean,scripts/noshake.json |
8 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
21-857 21 days ago |
21-857 21 days ago |
0-537 8 minutes |
23966 |
astrainfinita author:astrainfinita |
refactor: unbundle algebra from `{Seminormed, Normed}(Add)(Comm)Group` |
---
[](https://gitpod.io/from-referrer/)
- [ ] depends on: #23621
- [ ] depends on: #23961
|
slow-typeclass-synthesis
t-algebra
t-analysis
merge-conflict
blocked-by-other-PR
label:t-algebra$ |
3233/2752 |
Archive/Imo/Imo1998Q2.lean,Counterexamples/LinearOrderWithPosMulPosEqZero.lean,Mathlib/Algebra/Module/ZLattice/Basic.lean,Mathlib/Algebra/Module/ZLattice/Covolume.lean,Mathlib/Algebra/Order/Field/Canonical.lean,Mathlib/Algebra/Order/Field/Rat.lean,Mathlib/Algebra/Order/Floor/Ring.lean,Mathlib/Algebra/Order/GroupWithZero/Canonical.lean,Mathlib/Algebra/Order/GroupWithZero/Finset.lean,Mathlib/Algebra/Order/Hom/Monoid.lean,Mathlib/Algebra/Order/Nonneg/Field.lean,Mathlib/Algebra/Order/Nonneg/Ring.lean,Mathlib/Algebra/Order/Ring/Nat.lean,Mathlib/Analysis/Analytic/Basic.lean,Mathlib/Analysis/Analytic/CPolynomial.lean,Mathlib/Analysis/Analytic/CPolynomialDef.lean,Mathlib/Analysis/Analytic/ChangeOrigin.lean,Mathlib/Analysis/Analytic/Composition.lean,Mathlib/Analysis/Analytic/Constructions.lean,Mathlib/Analysis/Analytic/Inverse.lean,Mathlib/Analysis/Analytic/IsolatedZeros.lean,Mathlib/Analysis/Analytic/IteratedFDeriv.lean,Mathlib/Analysis/Analytic/Linear.lean,Mathlib/Analysis/Analytic/Order.lean,Mathlib/Analysis/Analytic/Polynomial.lean,Mathlib/Analysis/Analytic/RadiusLiminf.lean,Mathlib/Analysis/Analytic/Uniqueness.lean,Mathlib/Analysis/Analytic/Within.lean,Mathlib/Analysis/Asymptotics/AsymptoticEquivalent.lean,Mathlib/Analysis/Asymptotics/Defs.lean,Mathlib/Analysis/Asymptotics/Lemmas.lean,Mathlib/Analysis/Asymptotics/SpecificAsymptotics.lean,Mathlib/Analysis/Asymptotics/TVS.lean,Mathlib/Analysis/Asymptotics/Theta.lean,Mathlib/Analysis/BoundedVariation.lean,Mathlib/Analysis/BoxIntegral/Basic.lean,Mathlib/Analysis/BoxIntegral/DivergenceTheorem.lean,Mathlib/Analysis/BoxIntegral/Integrability.lean,Mathlib/Analysis/BoxIntegral/Partition/Additive.lean,Mathlib/Analysis/BoxIntegral/Partition/Measure.lean,Mathlib/Analysis/CStarAlgebra/Basic.lean,Mathlib/Analysis/CStarAlgebra/CStarMatrix.lean,Mathlib/Analysis/CStarAlgebra/ContinuousLinearMap.lean,Mathlib/Analysis/CStarAlgebra/Matrix.lean,Mathlib/Analysis/CStarAlgebra/Module/Constructions.lean,Mathlib/Analysis/CStarAlgebra/Module/Defs.lean,Mathlib/Analysis/Calculus/AddTorsor/AffineMap.lean,Mathlib/Analysis/Calculus/AddTorsor/Coord.lean,Mathlib/Analysis/Calculus/BumpFunction/Basic.lean,Mathlib/Analysis/Calculus/BumpFunction/Convolution.lean,Mathlib/Analysis/Calculus/BumpFunction/FiniteDimension.lean,Mathlib/Analysis/Calculus/BumpFunction/InnerProduct.lean,Mathlib/Analysis/Calculus/BumpFunction/Normed.lean,Mathlib/Analysis/Calculus/Conformal/InnerProduct.lean,Mathlib/Analysis/Calculus/Conformal/NormedSpace.lean,Mathlib/Analysis/Calculus/ContDiff/Basic.lean,Mathlib/Analysis/Calculus/ContDiff/Bounds.lean,Mathlib/Analysis/Calculus/ContDiff/CPolynomial.lean,Mathlib/Analysis/Calculus/ContDiff/Defs.lean,Mathlib/Analysis/Calculus/ContDiff/FTaylorSeries.lean,Mathlib/Analysis/Calculus/ContDiff/FaaDiBruno.lean,Mathlib/Analysis/Calculus/ContDiff/FiniteDimension.lean,Mathlib/Analysis/Calculus/ContDiff/Operations.lean,Mathlib/Analysis/Calculus/ContDiff/RCLike.lean,Mathlib/Analysis/Calculus/ContDiff/WithLp.lean,Mathlib/Analysis/Calculus/DSlope.lean,Mathlib/Analysis/Calculus/Deriv/Abs.lean,Mathlib/Analysis/Calculus/Deriv/Add.lean,Mathlib/Analysis/Calculus/Deriv/AffineMap.lean,Mathlib/Analysis/Calculus/Deriv/Basic.lean,Mathlib/Analysis/Calculus/Deriv/Comp.lean,Mathlib/Analysis/Calculus/Deriv/Inv.lean,Mathlib/Analysis/Calculus/Deriv/Inverse.lean,Mathlib/Analysis/Calculus/Deriv/Linear.lean,Mathlib/Analysis/Calculus/Deriv/Mul.lean,Mathlib/Analysis/Calculus/Deriv/Prod.lean,Mathlib/Analysis/Calculus/Deriv/Shift.lean,Mathlib/Analysis/Calculus/Deriv/Slope.lean,Mathlib/Analysis/Calculus/Deriv/Star.lean,Mathlib/Analysis/Calculus/Deriv/Support.lean,Mathlib/Analysis/Calculus/Deriv/ZPow.lean,Mathlib/Analysis/Calculus/DiffContOnCl.lean,Mathlib/Analysis/Calculus/FDeriv/Add.lean,Mathlib/Analysis/Calculus/FDeriv/Analytic.lean,Mathlib/Analysis/Calculus/FDeriv/Basic.lean,Mathlib/Analysis/Calculus/FDeriv/Bilinear.lean,Mathlib/Analysis/Calculus/FDeriv/Comp.lean,Mathlib/Analysis/Calculus/FDeriv/Equiv.lean,Mathlib/Analysis/Calculus/FDeriv/Extend.lean,Mathlib/Analysis/Calculus/FDeriv/Linear.lean,Mathlib/Analysis/Calculus/FDeriv/Measurable.lean,Mathlib/Analysis/Calculus/FDeriv/Mul.lean,Mathlib/Analysis/Calculus/FDeriv/Norm.lean,Mathlib/Analysis/Calculus/FDeriv/Pi.lean,Mathlib/Analysis/Calculus/FDeriv/Prod.lean,Mathlib/Analysis/Calculus/FDeriv/RestrictScalars.lean,Mathlib/Analysis/Calculus/FDeriv/Star.lean,Mathlib/Analysis/Calculus/FDeriv/Symmetric.lean,Mathlib/Analysis/Calculus/FDeriv/WithLp.lean,Mathlib/Analysis/Calculus/FormalMultilinearSeries.lean |
579 |
7 |
['astrainfinita', 'github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
20-81323 20 days ago |
154-16873 5 months ago* |
0-0 0 seconds* |
22771 |
alreadydone author:alreadydone |
feat(Homotopy/Lifting): monodromy of covering maps and lifting criterion |
Define the monodromy of a covering map: given a path in the base space, lifting it through the covering map induces a bijection between the fibers at the two endpoints of the path. Definition 2.1 in https://ncatlab.org/nlab/show/monodromy.
---
- [ ] depends on: #28234
- [x] depends on: #22649
[](https://gitpod.io/from-referrer/)
|
t-algebraic-topology
blocked-by-other-PR
|
193/146 |
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 |
5 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
PatrickMassot assignee:PatrickMassot |
20-77108 20 days ago |
20-83630 20 days ago |
144-35711 144 days |
27364 |
101damnations author:101damnations |
feat(RepresentationTheory/Homological/GroupCohomology): cohomology of finite cyclic groups |
Let `k` be a commutative ring, `G` a group and `A` a `k`-linear `G`-representation. Given endomorphisms `φ, ψ : A ⟶ A` such that `φ ∘ ψ = ψ ∘ φ = 0`. Denote by `Chains(A, φ, ψ)` the periodic chain complex `... ⟶ A --φ--> A --ψ--> A --φ--> A --ψ--> A ⟶ 0` and by `Cochains(A, φ, ψ)` the periodic cochain complex `0 ⟶ A --ψ--> A --φ--> A --ψ--> A --φ--> A ⟶ ...`.
When `G` is finite and generated by `g : G`, then `P := Chains(k[G], N, ρ(g) - Id)` (with `ρ` the left regular representation) is a projective resolution of `k` as a trivial representation. In this PR we show that for `A : Rep k G`, `Hom(P, A)` is isomorphic to
`Cochains(A, N, ρ_A(g) - Id)` as a complex of `k`-modules, and hence the cohomology of this complex computes group cohomology.
---
- [ ] depends on: #27362
- [ ] depends on: #27361
- [ ] depends on: #27363
[](https://gitpod.io/from-referrer/)
|
t-algebra
blocked-by-other-PR
label:t-algebra$ |
364/0 |
Mathlib.lean,Mathlib/RepresentationTheory/Homological/FiniteCyclic.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/FiniteCyclic.lean,Mathlib/RepresentationTheory/Invariants.lean |
4 |
4 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
20-67888 20 days ago |
20-67888 20 days ago |
0-731 12 minutes |
27365 |
101damnations author:101damnations |
feat(RepresentationTheory/Homological/GroupHomology): homology of finite cyclic groups |
Let `k` be a commutative ring, `G` a group and `A` a `k`-linear `G`-representation. Given endomorphisms `φ, ψ : A ⟶ A` such that `φ ∘ ψ = ψ ∘ φ = 0`. Denote by `Chains(A, φ, ψ)` the periodic chain complex `... ⟶ A --φ--> A --ψ--> A --φ--> A --ψ--> A ⟶ 0`.
When `G` is finite and generated by `g : G`, then `P := Chains(k[G], N, ρ(g) - Id)` (with `ρ` the left regular representation) is a projective resolution of `k` as a trivial representation.
In this PR we show that for `A : Rep k G`, `(A ⊗ P)_G` is isomorphic to `Chains(A, N, ρ_A(g) - Id)` as a complex of `k`-modules, and hence the homology of this complex computes group homology.
---
- [ ] depends on: #27362
- [ ] depends on: #27361
- [ ] depends on: #27363
[](https://gitpod.io/from-referrer/)
|
t-algebra
blocked-by-other-PR
label:t-algebra$ |
364/0 |
Mathlib.lean,Mathlib/RepresentationTheory/Homological/FiniteCyclic.lean,Mathlib/RepresentationTheory/Homological/GroupHomology/FiniteCyclic.lean,Mathlib/RepresentationTheory/Invariants.lean |
4 |
4 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
20-67883 20 days ago |
20-67883 20 days ago |
0-606 10 minutes |
27366 |
101damnations author:101damnations |
feat(RepresentationTheory/Homological/GroupCohomology/Hilbert90): add Hilbert 90 for cyclic groups |
Let `L/K` be a finite extension of fields. Before this PR, this file proves Noether's generalization of Hilbert's Theorem 90: that the 1st group cohomology $H^1(Aut_K(L), L^\times)$ is trivial.
Hilbert's original statement was that if $L/K$ is Galois, and $Gal(L/K)$ is cyclic, generated by an element `σ`, then for every `x : L` such that $N_{L/K}(x) = 1,$ there exists `y : L` such that $x = y/σ(y).$ We prove that in this PR, using the fact that `H¹(G, A) ≅ Ker(N_A)/(ρ(g) - 1)(A)` for any finite cyclic group `G` with generator `g`, and then applying Noether's generalization.
---
- [ ] depends on: #27361
- [ ] depends on: #27362
- [ ] depends on: #27363
- [ ] depends on: #27364
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebra
merge-conflict
blocked-by-other-PR
label:t-algebra$ |
417/8 |
Mathlib.lean,Mathlib/CategoryTheory/Action/Limits.lean,Mathlib/RepresentationTheory/Homological/FiniteCyclic.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/FiniteCyclic.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/Hilbert90.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/LowDegree.lean,Mathlib/RepresentationTheory/Invariants.lean,Mathlib/RepresentationTheory/Rep.lean |
8 |
4 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
20-67878 20 days ago |
20-67878 20 days ago |
0-351 5 minutes |
28808 |
alreadydone author:alreadydone |
experiment: Ideal with Mul only (no Semiring) |
---
- [ ] depends on: #28807
[](https://gitpod.io/from-referrer/)
|
bench-after-CI
t-algebra
awaiting-CI
blocked-by-other-PR
label:t-algebra$ |
172/120 |
Mathlib/Algebra/Module/Submodule/Defs.lean,Mathlib/Algebra/Module/Submodule/Lattice.lean,Mathlib/LinearAlgebra/Matrix/Ideal.lean,Mathlib/LinearAlgebra/TensorProduct/Subalgebra.lean,Mathlib/RingTheory/AdicCompletion/Basic.lean,Mathlib/RingTheory/DividedPowers/SubDPIdeal.lean,Mathlib/RingTheory/Ideal/Defs.lean,Mathlib/RingTheory/Ideal/Lattice.lean,Mathlib/RingTheory/PrincipalIdealDomain.lean,Mathlib/RingTheory/Spectrum/Prime/RingHom.lean |
10 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
20-62247 20 days ago |
20-73314 20 days ago |
0-0 0 seconds |
28700 |
Timeroot author:Timeroot |
feat(ModelTheory): Set.Definable is transitive |
---
This PR continues the work from #19695.
Original PR: https://github.com/leanprover-community/mathlib4/pull/19695
- [ ] depends on: #26332
[](https://gitpod.io/from-referrer/)
|
large-import
t-logic
blocked-by-other-PR
|
529/8 |
Mathlib/Data/Rel.lean,Mathlib/ModelTheory/Definability.lean,Mathlib/ModelTheory/Semantics.lean,Mathlib/ModelTheory/Syntax.lean,scripts/noshake.json |
5 |
4 |
['Timeroot', 'github-actions', 'mathlib4-dependent-issues-bot', 'staroperator'] |
nobody |
20-49218 20 days ago |
20-49219 20 days ago |
3-12935 3 days |
28787 |
alreadydone author:alreadydone |
feat(Counterexamples): a domain whose ring of differences is not a domain |
Example produced by Gemini 2.5 Pro: https://gemini.google.com/share/9558539e1309
---
- [ ] depends on: #28468
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebra
merge-conflict
blocked-by-other-PR
label:t-algebra$ |
1200/204 |
Counterexamples.lean,Counterexamples/GrothendieckAddGroupIsDomain.lean,Mathlib.lean,Mathlib/Algebra/Group/Subsemigroup/Defs.lean,Mathlib/Algebra/Module/End.lean,Mathlib/Algebra/Module/LocalizedModule/IsLocalization.lean,Mathlib/Algebra/Order/Nonneg/Basic.lean,Mathlib/Algebra/Order/Nonneg/Ring.lean,Mathlib/Algebra/Ring/Invertible.lean,Mathlib/GroupTheory/MonoidLocalization/Archimedean.lean,Mathlib/GroupTheory/MonoidLocalization/Basic.lean,Mathlib/GroupTheory/MonoidLocalization/Lemmas.lean,Mathlib/GroupTheory/MonoidLocalization/MonoidWithZero.lean,Mathlib/LinearAlgebra/TensorProduct/Basic.lean,Mathlib/RingTheory/IsTensorProduct.lean,Mathlib/RingTheory/Localization/Additive.lean,Mathlib/RingTheory/Localization/Away/Basic.lean,Mathlib/RingTheory/Localization/Basic.lean,Mathlib/RingTheory/Localization/Defs.lean,Mathlib/RingTheory/Localization/Ideal.lean,Mathlib/RingTheory/Localization/StrongRankCondition.lean,Mathlib/RingTheory/Smooth/StandardSmooth.lean,Mathlib/RingTheory/Trace/Quotient.lean |
23 |
6 |
['alreadydone', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'riccardobrasca'] |
nobody |
19-71145 19 days ago |
19-71145 19 days ago |
1-48447 1 day |
23920 |
YaelDillies author:YaelDillies |
feat: relation-separated sets |
Define a notion of separation of a set relative to a relation. This will be used to unify metric and dynamical separation.
From MiscYD and LeanAPAP
---
- [ ] depends on: #26988
[](https://gitpod.io/from-referrer/)
|
t-data
blocked-by-other-PR
|
248/8 |
Mathlib.lean,Mathlib/Combinatorics/SimpleGraph/Basic.lean,Mathlib/Data/Rel.lean,Mathlib/Data/Rel/Separated.lean |
4 |
20 |
['ADedecker', 'D-Thomine', 'YaelDillies', 'b-mehta', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
ADedecker assignee:ADedecker |
19-17698 19 days ago |
31-14630 1 month ago |
30-63957 30 days |
28475 |
astrainfinita author:astrainfinita |
chore(Analysis/SpecificLimits/Basic): generalize lemmas |
---
- [ ] depends on: #28472
- [ ] depends on: #28474
[](https://gitpod.io/from-referrer/)
|
t-analysis
merge-conflict
blocked-by-other-PR
|
131/98 |
Mathlib/Analysis/Normed/Algebra/Exponential.lean,Mathlib/Analysis/SpecificLimits/Basic.lean,Mathlib/Analysis/SpecificLimits/RCLike.lean,Mathlib/Data/Real/Hyperreal.lean,Mathlib/Topology/Algebra/Order/Field.lean,Mathlib/Topology/Instances/Rat.lean |
6 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
17-74620 17 days ago |
17-74621 17 days ago |
0-2105 35 minutes |
27578 |
bjornsolheim author:bjornsolheim |
feat(Geometry/Convex/Cone): add conical combinations and conical hull |
- Prove closure properties of sequences with nonnegative coefficients
- Define conical hull
- Prove that the smallest pointed cone containing s is the conical hull of s
- Implemented with Finsupp
---
- [ ] depends on: #25292
[](https://gitpod.io/from-referrer/)
|
t-convex-geometry
new-contributor
blocked-by-other-PR
|
188/0 |
Mathlib.lean,Mathlib/Geometry/Convex/Cone/ConicalHull.lean |
2 |
8 |
['YaelDillies', 'bjornsolheim', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
17-65294 17 days ago |
31-60994 1 month ago |
0-254 4 minutes |
28596 |
CBirkbeck author:CBirkbeck |
Dedekind eta e2 |
We show that the logarithmic derivative of the Dedekind eta function equals the the Eisenstein series E2 (up to a constant).
---
- [ ] depends on: #27606
- [ ] depends on: #26014
- [x] depends on: #28400
[](https://gitpod.io/from-referrer/)
|
large-import
merge-conflict
blocked-by-other-PR
|
1236/22 |
Mathlib.lean,Mathlib/Analysis/Asymptotics/Lemmas.lean,Mathlib/Analysis/Calculus/Deriv/Basic.lean,Mathlib/Analysis/Calculus/LogDeriv.lean,Mathlib/Analysis/Calculus/LogDerivUniformlyOn.lean,Mathlib/Analysis/Complex/Exponential.lean,Mathlib/Analysis/Complex/IntegerCompl.lean,Mathlib/Analysis/Complex/SummableUniformlyOn.lean,Mathlib/Analysis/Normed/Module/FiniteDimension.lean,Mathlib/Analysis/SpecialFunctions/Log/Summable.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Cotangent.lean,Mathlib/NumberTheory/ArithmeticFunction.lean,Mathlib/NumberTheory/LSeries/RiemannZeta.lean,Mathlib/NumberTheory/ModularForms/DedekindEta.lean,Mathlib/NumberTheory/ModularForms/EisensteinSeries/Defs.lean,Mathlib/NumberTheory/ModularForms/EisensteinSeries/E2.lean,Mathlib/NumberTheory/ModularForms/EisensteinSeries/QExpansion.lean,Mathlib/NumberTheory/ModularForms/EisensteinSeries/Summable.lean,Mathlib/NumberTheory/TsumDivsorsAntidiagonal.lean,Mathlib/RingTheory/EuclideanDomain.lean,Mathlib/Topology/Algebra/InfiniteSum/Basic.lean,Mathlib/Topology/Algebra/InfiniteSum/NatInt.lean |
22 |
n/a |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
15-74834 15 days ago |
unknown |
unknown |
28685 |
mitchell-horner author:mitchell-horner |
feat(Combinatorics/SimpleGraph): prove the minimal-degree version of the Erdős-Stone theorem |
Proves the minimal degree-version of the Erdős-Stone theorem:
If `G` has a minimal degree of at least `(1 - 1 / r + o(1)) * card V`, then `G` contains a copy of a `completeEquipartiteGraph` in `r + 1` parts each of size `t`.
The double-counting construction from the proof is available in `namespace ErdosStone`.
---
- [ ] depends on: #25843
- [x] depends on: #27597
- [ ] depends on: #27599
- [x] depends on: #28443
- [ ] depends on: #28445
- [x] depends on: #28446
- [x] depends on: #28447
Similar to #25841 I've tried to make as much of the double-counting construction *not* private as possible. I figure it is useful to borrow constructions between proofs.
If this is just considered garbage and bloat and better left private. Please let me know.
[](https://gitpod.io/from-referrer/)
|
t-combinatorics
merge-conflict
blocked-by-other-PR
WIP
|
582/14 |
Mathlib.lean,Mathlib/Combinatorics/SimpleGraph/Bipartite.lean,Mathlib/Combinatorics/SimpleGraph/CompleteMultipartite.lean,Mathlib/Combinatorics/SimpleGraph/Extremal/Basic.lean,Mathlib/Combinatorics/SimpleGraph/Extremal/ErdosStoneSimonovits.lean,Mathlib/Combinatorics/SimpleGraph/Finite.lean,Mathlib/Combinatorics/SimpleGraph/Maps.lean,Mathlib/Combinatorics/SimpleGraph/Operations.lean,Mathlib/Data/Finset/Union.lean,Mathlib/Data/Nat/Cast/Order/Field.lean |
10 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
15-74710 15 days ago |
15-74711 15 days ago |
0-46 46 seconds |
28686 |
mitchell-horner author:mitchell-horner |
feat(Combinatorics/SimpleGraph): prove the Erdős-Stone theorem |
Proves the Erdős-Stone theorem:
If `G` has at least `(1 - 1 / r + o(1)) * card V ^ 2 / 2` many edges, then `G` contains a copy of a `completeEquipartiteGraph (r + 1) t`.
---
- [ ] depends on: #28685
[](https://gitpod.io/from-referrer/)
|
t-combinatorics
merge-conflict
blocked-by-other-PR
WIP
|
757/14 |
Mathlib.lean,Mathlib/Combinatorics/SimpleGraph/Bipartite.lean,Mathlib/Combinatorics/SimpleGraph/CompleteMultipartite.lean,Mathlib/Combinatorics/SimpleGraph/Extremal/Basic.lean,Mathlib/Combinatorics/SimpleGraph/Extremal/ErdosStoneSimonovits.lean,Mathlib/Combinatorics/SimpleGraph/Finite.lean,Mathlib/Combinatorics/SimpleGraph/Maps.lean,Mathlib/Combinatorics/SimpleGraph/Operations.lean,Mathlib/Data/Finset/Union.lean,Mathlib/Data/Nat/Cast/Order/Field.lean |
10 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
15-74708 15 days ago |
15-74709 15 days ago |
0-10 10 seconds |
28687 |
mitchell-horner author:mitchell-horner |
feat(Combinatorics/SimpleGraph): prove the Erdős-Stone-Simonovits theorem |
Proves the Erdős-Stone-Simonovits theorem:
If the chromatic number of `H` equals `r + 1 > 0`, then the `extremalNumber` of `H` is greater than `(1 - 1 / r - o(1)) * card V ^ 2 / 2` and at most `(1 - 1 / r + o(1)) * card V ^ 2 / 2`.
---
- [ ] depends on: #28686
[](https://gitpod.io/from-referrer/)
|
t-combinatorics
merge-conflict
blocked-by-other-PR
WIP
|
879/14 |
Mathlib.lean,Mathlib/Combinatorics/SimpleGraph/Bipartite.lean,Mathlib/Combinatorics/SimpleGraph/CompleteMultipartite.lean,Mathlib/Combinatorics/SimpleGraph/Extremal/Basic.lean,Mathlib/Combinatorics/SimpleGraph/Extremal/ErdosStoneSimonovits.lean,Mathlib/Combinatorics/SimpleGraph/Finite.lean,Mathlib/Combinatorics/SimpleGraph/Maps.lean,Mathlib/Combinatorics/SimpleGraph/Operations.lean,Mathlib/Data/Finset/Union.lean,Mathlib/Data/Nat/Cast/Order/Field.lean |
10 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
15-74707 15 days ago |
15-74708 15 days ago |
0-74 1 minute |
28689 |
mitchell-horner author:mitchell-horner |
feat(Combinatorics/SimpleGraph): prove well-known corollaries of the Erdős-Stone-Simonovits theorem |
Proves well-known corollaries of the Erdős-Stone-Simonovits theorem:
E.g., if the chromatic number of `H` equals `r + 1 > 1`, then `extremalNumber n H` is asymptotically equivalent to `(1 - 1 / r) * n.choose 2` as `n → ∞`
---
- [ ] depends on: #28687
[](https://gitpod.io/from-referrer/)
|
t-combinatorics
merge-conflict
blocked-by-other-PR
WIP
|
958/14 |
Mathlib.lean,Mathlib/Combinatorics/SimpleGraph/Bipartite.lean,Mathlib/Combinatorics/SimpleGraph/CompleteMultipartite.lean,Mathlib/Combinatorics/SimpleGraph/Extremal/Basic.lean,Mathlib/Combinatorics/SimpleGraph/Extremal/ErdosStoneSimonovits.lean,Mathlib/Combinatorics/SimpleGraph/Finite.lean,Mathlib/Combinatorics/SimpleGraph/Maps.lean,Mathlib/Combinatorics/SimpleGraph/Operations.lean,Mathlib/Data/Finset/Union.lean,Mathlib/Data/Nat/Cast/Order/Field.lean |
10 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
15-74706 15 days ago |
15-74707 15 days ago |
0-45 45 seconds |
23460 |
Timeroot author:Timeroot |
feat: Definition of `Clone` |
Basics about Clones. Part of #20051
---
- [ ] depends on: #26329
[](https://gitpod.io/from-referrer/)
|
t-algebra
blocked-by-other-PR
label:t-algebra$ |
326/0 |
Mathlib.lean,Mathlib/Algebra/Clone/Basic.lean,Mathlib/Algebra/Clone/Defs.lean,Mathlib/Data/Fin/Basic.lean |
4 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
dagurtomas assignee:dagurtomas |
15-59684 15 days ago |
15-59685 15 days ago |
65-54988 65 days |
29076 |
yury-harmonic author:yury-harmonic |
feat(BigOperators/ModEq): new file |
---
- [ ] depends on: #29072
[](https://gitpod.io/from-referrer/)
|
blocked-by-other-PR |
319/15 |
Mathlib.lean,Mathlib/Algebra/BigOperators/ModEq.lean,Mathlib/Data/Int/ModEq.lean,Mathlib/Data/Nat/ModEq.lean |
4 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
15-53127 15 days ago |
15-59965 15 days ago |
0-726 12 minutes |
26890 |
robin-carlier author:robin-carlier |
feat(CategoryTheory/Monoidal/DayConvolution) : more API for `DayFunctor` |
We provide some lemmas that helps characterizing the monoidal structure on `DayFunctor`, they are special cases of the lemmas for `LawfulDayConvolutionMonoidalCategoryStruct`.
---
- [ ] depends on: #26824
[](https://gitpod.io/from-referrer/)
|
t-category-theory
merge-conflict
blocked-by-other-PR
|
1372/19 |
Mathlib.lean,Mathlib/CategoryTheory/Functor/KanExtension/Basic.lean,Mathlib/CategoryTheory/Monoidal/DayConvolution.lean,Mathlib/CategoryTheory/Monoidal/DayConvolution/DayFunctor.lean |
4 |
n/a |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
15-46919 15 days ago |
unknown |
unknown |
26952 |
robin-carlier author:robin-carlier |
feat(CategoryTheory/DayConvolution): monoid objects internal to day convolutions |
In this file, given `F : C ⊛⥤ V`, we provide a bijective correspondence between lax monoidal structures on `F.functor` and
`Mon_Class F` structures. We also prove that through this correspondance, monoidal natural transformations correspond to morphisms of internal monoid objects.
---
- [ ] depends on: #26890
[](https://gitpod.io/from-referrer/)
|
t-category-theory
merge-conflict
blocked-by-other-PR
|
1574/19 |
Mathlib.lean,Mathlib/CategoryTheory/Functor/KanExtension/Basic.lean,Mathlib/CategoryTheory/Monoidal/DayConvolution.lean,Mathlib/CategoryTheory/Monoidal/DayConvolution/DayFunctor.lean,Mathlib/CategoryTheory/Monoidal/DayConvolution/Mon_.lean |
5 |
5 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
15-46917 15 days ago |
15-46918 15 days ago |
0-584 9 minutes |
27133 |
robin-carlier author:robin-carlier |
feat(CategoryTheory/Monoidal/DayConvolution): `C ⊛⥤ V` is monoidal closed when `V` is |
When `V` is a monoidal closed category admitting enough limits, we show that the type alias `C ⊛⥤ V` for functors `C ⥤ V` with Day convolution monoidal structure is monoidal closed using the API for `LawfulDayConvolutionClosedMonoidalCategoryStruct` developped in #27119.
We expose the required data to exhibit (realization as a functor of) the internal hom as a suitable, and we port the lemmas that characterize its functoriality in that regard, as well as the evaluation and coevaluation morphisms.
---
- [ ] depends on: #27119
- [ ] depends on: #26890
[](https://gitpod.io/from-referrer/)
|
t-category-theory
merge-conflict
blocked-by-other-PR
|
1706/20 |
Mathlib.lean,Mathlib/CategoryTheory/Functor/KanExtension/Basic.lean,Mathlib/CategoryTheory/Monoidal/DayConvolution.lean,Mathlib/CategoryTheory/Monoidal/DayConvolution/Closed.lean,Mathlib/CategoryTheory/Monoidal/DayConvolution/DayFunctor.lean |
5 |
n/a |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
15-46792 15 days ago |
unknown |
unknown |
27151 |
robin-carlier author:robin-carlier |
feat(CategoryTheory/Monoidal/DayConvolution): `C ⊛⥤ V` is braided/symmetric when `C` and `V` are braided/symmetric |
We use the machinery from #27150 to show that Day functors (the type alias for functors endowed with the Day convolution monoidal structure) are braided/symmetric when the base categories are.
---
- [ ] depends on: #27150
- [ ] depends on: #26890
[](https://gitpod.io/from-referrer/)
|
t-category-theory
merge-conflict
blocked-by-other-PR
|
1591/20 |
Mathlib.lean,Mathlib/CategoryTheory/Functor/KanExtension/Basic.lean,Mathlib/CategoryTheory/Monoidal/DayConvolution.lean,Mathlib/CategoryTheory/Monoidal/DayConvolution/Braided.lean,Mathlib/CategoryTheory/Monoidal/DayConvolution/DayFunctor.lean |
5 |
n/a |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
15-46790 15 days ago |
unknown |
unknown |
27175 |
robin-carlier author:robin-carlier |
feat(CategoryTheory/Monoidal/DayConvolution): `LawfulDayConvolutionMonoidalCategoryStruct.ι C V D` is monoidal when the target is `C ⊛⥤ V` |
We prove a "soundness" result for our notion of `LawfulDayConvolutionMonoidalCategoryStruct`, i.e that when be interpret its field `ι` as valued in Day functors (the type alias for functors endowed with the Day convolution monoidal structure), the data from `LawfulDayConvolutionMonoidalCategoryStruct` turn `ι` in a monoidal functor, proving that the categories endowed with such a structure are precisely those that can be identified to monoidal (not necessarily full) subcategories of Day functors.
Implicitly, the structure isomorphisms for this monoidal structure bundle isomorphisms asserting unicity up to isomorphisms of day convolutions.
---
- [ ] depends on: #26890
[](https://gitpod.io/from-referrer/)
|
t-category-theory
merge-conflict
blocked-by-other-PR
|
1585/24 |
Mathlib.lean,Mathlib/CategoryTheory/Functor/KanExtension/Basic.lean,Mathlib/CategoryTheory/Monoidal/DayConvolution.lean,Mathlib/CategoryTheory/Monoidal/DayConvolution/DayFunctor.lean |
4 |
n/a |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
15-46789 15 days ago |
unknown |
unknown |
29080 |
vihdzp author:vihdzp |
feat: `Colex` order on pi types |
We define an order instance on `Colex (∀ i, β i)`, so that its `<` relation is `Pi.Lex (· > ·) (· < ·)`.
---
- [ ] depends on: #29058 (this PR should build after merging)
[](https://gitpod.io/from-referrer/)
|
t-order
blocked-by-other-PR
|
157/12 |
Mathlib/Order/PiLex.lean,Mathlib/Order/Synonym.lean |
2 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
15-29687 15 days ago |
15-54665 15 days ago |
0-456 7 minutes |
23181 |
YaelDillies author:YaelDillies |
refactor(Topology/UniformSpace): use `SetRel` |
What's left in `UniformSpace.Defs` is precisely the theory of the uniformity filter.
The motivation is that the theory of coverings and packings in both high dimensional probability and dynamics can be based on entourages, while they have little to do with the uniformity filter (indeed, entourages are in a sense a quantitative version of the uniformity filter).
---
- [x] depends on: #25587
- [ ] depends on: #26988
[](https://gitpod.io/from-referrer/)
|
t-topology
blocked-by-other-PR
|
807/609 |
Mathlib/Combinatorics/SimpleGraph/Basic.lean,Mathlib/Data/Rel.lean,Mathlib/Dynamics/TopologicalEntropy/CoverEntropy.lean,Mathlib/Dynamics/TopologicalEntropy/DynamicalEntourage.lean,Mathlib/Dynamics/TopologicalEntropy/NetEntropy.lean,Mathlib/Dynamics/TopologicalEntropy/Semiconj.lean,Mathlib/Dynamics/TopologicalEntropy/Subset.lean,Mathlib/InformationTheory/Hamming.lean,Mathlib/MeasureTheory/Measure/RegularityCompacts.lean,Mathlib/Topology/MetricSpace/BundledFun.lean,Mathlib/Topology/MetricSpace/PiNat.lean,Mathlib/Topology/Metrizable/Uniformity.lean,Mathlib/Topology/UniformSpace/Ascoli.lean,Mathlib/Topology/UniformSpace/Basic.lean,Mathlib/Topology/UniformSpace/Cauchy.lean,Mathlib/Topology/UniformSpace/Compact.lean,Mathlib/Topology/UniformSpace/CompactConvergence.lean,Mathlib/Topology/UniformSpace/Completion.lean,Mathlib/Topology/UniformSpace/Defs.lean,Mathlib/Topology/UniformSpace/DiscreteUniformity.lean,Mathlib/Topology/UniformSpace/Equicontinuity.lean,Mathlib/Topology/UniformSpace/HeineCantor.lean,Mathlib/Topology/UniformSpace/OfCompactT2.lean,Mathlib/Topology/UniformSpace/OfFun.lean,Mathlib/Topology/UniformSpace/Separation.lean,Mathlib/Topology/UniformSpace/Ultra/Basic.lean,Mathlib/Topology/UniformSpace/Ultra/Constructions.lean,Mathlib/Topology/UniformSpace/UniformApproximation.lean,Mathlib/Topology/UniformSpace/UniformConvergence.lean,Mathlib/Topology/UniformSpace/UniformEmbedding.lean |
30 |
34 |
['ADedecker', 'PatrickMassot', 'YaelDillies', 'b-mehta', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
14-12409 14 days ago |
14-12428 14 days ago |
75-62949 75 days |
23124 |
YaelDillies author:YaelDillies |
feat(MetricSpace): nets |
Define nets, which are a quantitative notion of compactness in a metric space.
From my PhD (MiscYD)
---
- [x] depends on: #23180
- [ ] depends on: #23181
- [ ] depends on: #23920
[](https://gitpod.io/from-referrer/)
|
t-topology
awaiting-CI
blocked-by-other-PR
|
1158/686 |
Mathlib.lean,Mathlib/Combinatorics/SimpleGraph/Basic.lean,Mathlib/Data/Rel.lean,Mathlib/Data/Rel/Cover.lean,Mathlib/Data/Rel/Separated.lean,Mathlib/Dynamics/TopologicalEntropy/CoverEntropy.lean,Mathlib/Dynamics/TopologicalEntropy/DynamicalEntourage.lean,Mathlib/Dynamics/TopologicalEntropy/NetEntropy.lean,Mathlib/Dynamics/TopologicalEntropy/Semiconj.lean,Mathlib/Dynamics/TopologicalEntropy/Subset.lean,Mathlib/InformationTheory/Hamming.lean,Mathlib/MeasureTheory/Measure/RegularityCompacts.lean,Mathlib/Topology/MetricSpace/BundledFun.lean,Mathlib/Topology/MetricSpace/Cover.lean,Mathlib/Topology/MetricSpace/MetricSeparated.lean,Mathlib/Topology/MetricSpace/PiNat.lean,Mathlib/Topology/Metrizable/Uniformity.lean,Mathlib/Topology/UniformSpace/Ascoli.lean,Mathlib/Topology/UniformSpace/Basic.lean,Mathlib/Topology/UniformSpace/Cauchy.lean,Mathlib/Topology/UniformSpace/Compact.lean,Mathlib/Topology/UniformSpace/CompactConvergence.lean,Mathlib/Topology/UniformSpace/Completion.lean,Mathlib/Topology/UniformSpace/Defs.lean,Mathlib/Topology/UniformSpace/DiscreteUniformity.lean,Mathlib/Topology/UniformSpace/Equicontinuity.lean,Mathlib/Topology/UniformSpace/HeineCantor.lean,Mathlib/Topology/UniformSpace/OfCompactT2.lean,Mathlib/Topology/UniformSpace/OfFun.lean,Mathlib/Topology/UniformSpace/Separation.lean,Mathlib/Topology/UniformSpace/Ultra/Basic.lean,Mathlib/Topology/UniformSpace/Ultra/Constructions.lean,Mathlib/Topology/UniformSpace/UniformApproximation.lean,Mathlib/Topology/UniformSpace/UniformConvergence.lean,Mathlib/Topology/UniformSpace/UniformEmbedding.lean |
35 |
20 |
['D-Thomine', 'YaelDillies', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'urkud'] |
nobody |
14-12353 14 days ago |
14-12377 14 days ago |
1-52822 1 day |
28819 |
ScottCarnahan author:ScottCarnahan |
feat (Data/Finsupp): define convolution smul for finsupps on formal functions |
This is a generalization of the multiplication action of the ring of Laurent polynomials on the space of formal power series with unbounded pole terms.
---
- [ ] depends on: #28876
[](https://gitpod.io/from-referrer/)
|
blocked-by-other-PR |
127/15 |
Mathlib.lean,Mathlib/Algebra/Group/Action/Defs.lean,Mathlib/Algebra/Order/AddTorsor.lean,Mathlib/Data/Finset/SMulAntidiagonal.lean,Mathlib/Data/Finsupp/PointwiseSMul.lean,Mathlib/Data/Set/SMulAntidiagonal.lean,Mathlib/RingTheory/HahnSeries/Multiplication.lean |
7 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
13-83992 13 days ago |
14-2986 14 days ago |
1-6093 1 day |
28893 |
joelriou author:joelriou |
refactor(AlgebraicTopology): redefine the topological simplex using the convexity API |
Before this PR, the n-dimensional topological simplex (in the `AlgebraicTopology` hierarchy) was defined as a subtype of `Fin (n + 1) → ℝ≥0`, which did not interact well with the convexity API which assumes the ambient type is a vector space. In this PR, we redefine the topological simplex functor (as a cosimplicial object in `TopCat`) using the already existing `stdSimplex` from `Analysis.Convex`.
---
- [ ] depends on: #28891
- [x] depends on: #28869
[](https://gitpod.io/from-referrer/)
|
t-algebraic-topology
t-convex-geometry
large-import
blocked-by-other-PR
|
283/109 |
Mathlib.lean,Mathlib/AlgebraicTopology/SimplexCategory/Basic.lean,Mathlib/AlgebraicTopology/SingularSet.lean,Mathlib/AlgebraicTopology/TopologicalSimplex.lean,Mathlib/Analysis/Convex/StdSimplex.lean,Mathlib/LinearAlgebra/Finsupp/Pi.lean,Mathlib/Topology/Algebra/Monoid/FunOnFinite.lean |
7 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
13-66442 13 days ago |
13-66591 13 days ago |
0-2609 43 minutes |
28013 |
astrainfinita author:astrainfinita |
feat: Lindemann-Weierstrass Theorem |
This PR continues the work from #6718.
--------
- [x] depends on: #18693
- [ ] depends on: #29121 |
t-algebra
t-analysis
merge-conflict
blocked-by-other-PR
WIP
label:t-algebra$ |
1205/53 |
Mathlib.lean,Mathlib/Algebra/MonoidAlgebra/Basic.lean,Mathlib/Algebra/Polynomial/Splits.lean,Mathlib/Data/Finsupp/Defs.lean,Mathlib/NumberTheory/Transcendental/Lindemann/AlgebraicPart.lean,Mathlib/NumberTheory/Transcendental/Lindemann/AnalyticalPart.lean,Mathlib/NumberTheory/Transcendental/Lindemann/Basic.lean,Mathlib/NumberTheory/Transcendental/Lindemann/SumAEvalARoots.lean,Mathlib/RingTheory/MvPolynomial/Symmetric/Eval.lean,docs/100.yaml,docs/1000.yaml |
11 |
n/a |
['astrainfinita', 'github-actions', 'j-loreaux', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
13-23584 13 days ago |
unknown |
unknown |
28962 |
grunweg author:grunweg |
chore: enable the flexible linter in mathlib |
Let's see what has regressed in the mean-time, and how many exceptions remain.
We're somewhat liberal with disabling the linter when this doesn't make sense: let's see how close we are.
---
TODO: should the `bicategory` tactic be considered flexible/normalising?
- [ ] depends on: #29027
- [ ] depends on: #29174
[](https://gitpod.io/from-referrer/)
|
merge-conflict
blocked-by-other-PR
|
613/203 |
Archive/Arithcc.lean,Archive/Examples/Eisenstein.lean,Archive/Examples/IfNormalization/Result.lean,Archive/Imo/Imo1997Q3.lean,Archive/Imo/Imo2008Q2.lean,Archive/Imo/Imo2008Q4.lean,Archive/Imo/Imo2019Q4.lean,Archive/Imo/Imo2024Q5.lean,Archive/Wiedijk100Theorems/CubingACube.lean,Counterexamples/MapFloor.lean,Counterexamples/Phillips.lean,Mathlib/Algebra/BigOperators/Fin.lean,Mathlib/Algebra/Category/ModuleCat/Subobject.lean,Mathlib/Algebra/Field/GeomSum.lean,Mathlib/Algebra/FreeAlgebra.lean,Mathlib/Algebra/Group/Submonoid/Basic.lean,Mathlib/Algebra/Homology/Augment.lean,Mathlib/Algebra/Lie/Nilpotent.lean,Mathlib/Algebra/Lie/Weights/RootSystem.lean,Mathlib/Algebra/LinearRecurrence.lean,Mathlib/Algebra/Polynomial/Bivariate.lean,Mathlib/Algebra/Ring/Subring/Basic.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Affine/Formula.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Affine/Point.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Jacobian/Formula.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Projective/Formula.lean,Mathlib/AlgebraicGeometry/Gluing.lean,Mathlib/AlgebraicGeometry/Limits.lean,Mathlib/AlgebraicGeometry/StructureSheaf.lean,Mathlib/AlgebraicGeometry/ValuativeCriterion.lean,Mathlib/AlgebraicTopology/SimplicialSet/HomotopyCat.lean,Mathlib/AlgebraicTopology/SimplicialSet/NerveAdjunction.lean,Mathlib/Analysis/Analytic/Binomial.lean,Mathlib/Analysis/Analytic/Constructions.lean,Mathlib/Analysis/Analytic/OfScalars.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Basic.lean,Mathlib/Analysis/CStarAlgebra/SpecialFunctions/PosPart.lean,Mathlib/Analysis/Calculus/ContDiff/FaaDiBruno.lean,Mathlib/Analysis/Calculus/FDeriv/Analytic.lean,Mathlib/Analysis/Calculus/FDeriv/Measurable.lean,Mathlib/Analysis/Calculus/FDeriv/Pow.lean,Mathlib/Analysis/Calculus/FormalMultilinearSeries.lean,Mathlib/Analysis/Calculus/LHopital.lean,Mathlib/Analysis/Complex/Arg.lean,Mathlib/Analysis/Complex/Exponential.lean,Mathlib/Analysis/Complex/ValueDistribution/FirstMainTheorem.lean,Mathlib/Analysis/Fourier/FourierTransformDeriv.lean,Mathlib/Analysis/FunctionalSpaces/SobolevInequality.lean,Mathlib/Analysis/InnerProductSpace/Rayleigh.lean,Mathlib/Analysis/MeanInequalities.lean,Mathlib/Analysis/Meromorphic/Basic.lean,Mathlib/Analysis/Meromorphic/NormalForm.lean,Mathlib/Analysis/Meromorphic/TrailingCoefficient.lean,Mathlib/Analysis/NormedSpace/MultipliableUniformlyOn.lean,Mathlib/Analysis/ODE/Gronwall.lean,Mathlib/Analysis/Real/Pi/Irrational.lean,Mathlib/Analysis/SpecialFunctions/BinaryEntropy.lean,Mathlib/Analysis/SpecialFunctions/ContinuousFunctionalCalculus/Rpow/IntegralRepresentation.lean,Mathlib/Analysis/SpecialFunctions/Gaussian/FourierTransform.lean,Mathlib/Analysis/SpecialFunctions/MulExpNegMulSq.lean,Mathlib/Analysis/SpecialFunctions/MulExpNegMulSqIntegral.lean,Mathlib/Analysis/SpecialFunctions/Pow/NNReal.lean,Mathlib/Analysis/SpecialFunctions/Pow/Real.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Arctan.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Basic.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Complex.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Inverse.lean,Mathlib/Analysis/SpecificLimits/Normed.lean,Mathlib/CategoryTheory/Bicategory/Adjunction/Mate.lean,Mathlib/CategoryTheory/Dialectica/Monoidal.lean,Mathlib/CategoryTheory/Galois/Basic.lean,Mathlib/CategoryTheory/Limits/Constructions/Equalizers.lean,Mathlib/CategoryTheory/Limits/Shapes/BinaryProducts.lean,Mathlib/CategoryTheory/Limits/Shapes/Equalizers.lean,Mathlib/CategoryTheory/Limits/Shapes/Grothendieck.lean,Mathlib/CategoryTheory/Limits/Shapes/Products.lean,Mathlib/CategoryTheory/Limits/VanKampen.lean,Mathlib/CategoryTheory/Monoidal/DayConvolution/Braided.lean,Mathlib/CategoryTheory/Products/Basic.lean,Mathlib/CategoryTheory/SmallObject/Construction.lean,Mathlib/Combinatorics/Additive/Corner/Roth.lean,Mathlib/Combinatorics/Additive/FreimanHom.lean,Mathlib/Combinatorics/Additive/SmallTripling.lean,Mathlib/Combinatorics/Additive/VerySmallDoubling.lean,Mathlib/Combinatorics/Enumerative/Composition.lean,Mathlib/Combinatorics/SetFamily/FourFunctions.lean,Mathlib/Combinatorics/SetFamily/KruskalKatona.lean,Mathlib/Combinatorics/SimpleGraph/ConcreteColorings.lean,Mathlib/Combinatorics/SimpleGraph/Connectivity/WalkDecomp.lean,Mathlib/Combinatorics/SimpleGraph/Regularity/Uniform.lean,Mathlib/Computability/Halting.lean,Mathlib/Computability/Partrec.lean,Mathlib/Computability/PartrecCode.lean,Mathlib/Computability/Primrec.lean,Mathlib/Computability/TMConfig.lean,Mathlib/Computability/TMToPartrec.lean,Mathlib/Control/EquivFunctor/Instances.lean,Mathlib/Data/Bool/Count.lean,Mathlib/Data/ENNReal/BigOperators.lean,Mathlib/Data/ENat/Basic.lean |
167 |
17 |
['github-actions', 'grunweg', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
12-62536 12 days ago |
12-62942 12 days ago |
0-2 2 seconds |
26221 |
grunweg author:grunweg |
Mr. Covariant Derivatives |
This PR is a work in progress, and will land in individual pieces. Some contributions include
- additional API for differentiability of vector bundle sections
- finite sums, differences and scalar products of smooth sections are smooth
- the same result for mdifferentiable
- add missing mdifferentiable congruence lemmas
- define smooth local frames of a vector bundle
- a general tensoriality criterion (to be cleaned up!)
- define covariant derivatives, proving their tensoriality and that convex combinations of these are covariant derivatives
- the classification of covariant derivatives over a trivial bundle
- additional API for the Lie bracket of vector fields: the product rule (one sorry left!), Lie bracket at zero vanishes
- torsion of a connection, torsion-free connections
- Gram-Schmidt procedure for sections of a Riemannian vector bundle
- orthonormal frames on a Riemannian vector bundle
- connections compatible with a metric; definition of the Levi-Civita connection
- in progress: existence and uniqueness of the Levi-Civita connection
- custom elaborators for sections in a vector bundle and for differentiability/smoothness in a mathlib (inferring the model with corners) --- experimental
More to come soon!
Joint work with @PatrickMassot; supported by the FMJH.
---
- [x] depends on: #26360
- [x] depends on: #26672
- [x] depends on: #26673
- [x] depends on: #26674
- [x] depends on: #26864 (more of a by-product)
- [x] depends on: #26865
- [x] depends on: #26866
- [ ] depends on: #26870
- [ ] depends on: #26871
- [x] depends on: #26671
- [x] depends on: #26676
- [x] depends on: #26677
- [x] depends on: #26678
- [x] depends on: #26686
- [x] depends on: #26687
- [x] depends on: #26688
- [x] depends on: #26702
- [x] depends on: #26709
- [x] depends on: #26734
- [ ] depends on: #26743 (still WIP)
- [x] depends on: #26894
- [x] depends on: #26921
- [x] depends on: #26922
- [x] depends on: #27020
- [ ] depends on: #27021
- [x] depends on: #27023
- [ ] depends on: #27024
- [ ] depends on: #27025
[](https://gitpod.io/from-referrer/)
|
t-differential-geometry
merge-conflict
blocked-by-other-PR
|
6595/37 |
Mathlib.lean,Mathlib/Analysis/InnerProductSpace/GramSchmidtOrtho.lean,Mathlib/Geometry/Manifold/CheatSheet.md,Mathlib/Geometry/Manifold/ContMDiff/Defs.lean,Mathlib/Geometry/Manifold/Elaborators.lean,Mathlib/Geometry/Manifold/PartitionOfUnity.lean,Mathlib/Geometry/Manifold/Riemannian/ExistsRiemannianMetric.lean,Mathlib/Geometry/Manifold/Traces.lean,Mathlib/Geometry/Manifold/VectorBundle/Basic.lean,Mathlib/Geometry/Manifold/VectorBundle/CovariantDerivative/Basic.lean,Mathlib/Geometry/Manifold/VectorBundle/CovariantDerivative/LeviCivita.lean,Mathlib/Geometry/Manifold/VectorBundle/CovariantDerivative/Torsion.lean,Mathlib/Geometry/Manifold/VectorBundle/GramSchmidtOrtho.lean,Mathlib/Geometry/Manifold/VectorBundle/LocalFrame.lean,Mathlib/Geometry/Manifold/VectorBundle/MDifferentiable.lean,Mathlib/Geometry/Manifold/VectorBundle/Misc.lean,Mathlib/Geometry/Manifold/VectorBundle/OrthonormalFrame.lean,Mathlib/Geometry/Manifold/VectorBundle/SmoothSection.lean,Mathlib/Geometry/Manifold/VectorBundle/Tensoriality.lean,Mathlib/Geometry/Manifold/VectorField/LieBracket.lean,Mathlib/Geometry/Manifold/VectorField/Pullback.lean,Mathlib/Util/PrintSorries.lean,MathlibTest/DifferentialGeometry/Elaborators.lean |
23 |
n/a |
['github-actions', 'grunweg', 'idontgetoutmuch', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
12-60595 12 days ago |
unknown |
unknown |
26413 |
michaellee94 author:michaellee94 |
feat(Analysis/ODE/MaximalSolution): Existence of maximal solutions for ODE meeting Picard-Lindelöf conditions |
Add existence proof for maximal solution of ODE using Picard-Lindelöf and a uniqueness theorem using Grönwall's lemma.
---
- [x] depends on: #26382
- [ ] depends on: #29186
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-analysis
merge-conflict
awaiting-author
blocked-by-other-PR
|
746/1 |
Mathlib.lean,Mathlib/Analysis/ODE/MaximalSolution.lean,docs/undergrad.yaml |
3 |
13 |
['github-actions', 'grunweg', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'winstonyin'] |
nobody |
12-51524 12 days ago |
12-51525 12 days ago |
0-5139 1 hour |
29203 |
Hagb author:Hagb |
(WIP) feat(RingTheory/MvPolynomial/Groebner) : Gröbner basis |
WIP
Co-authored-by: Hao Shen [3118181069@qq.com](mailto:3118181069@qq.com)
---
CC @tsuki8
- [ ] depends on: #26039
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
large-import
blocked-by-other-PR
|
507/3 |
Mathlib/RingTheory/MvPolynomial/Groebner.lean,Mathlib/RingTheory/MvPolynomial/MonomialOrder.lean |
2 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
12-4828 12 days ago |
12-4829 12 days ago |
0-0 0 seconds |
28462 |
joelriou author:joelriou |
feat(AlgebraicTopology/SimplicialSet): the relative cell complex attached to a rank function for a pairing |
---
- [ ] depends on: #28351
- [ ] depends on: #28346
- [ ] depends on: #28336
- [ ] depends on: #28332
- [ ] depends on: #28330
- [ ] depends on: #28224
- [x] depends on: #27968
- [ ] depends on: #28034
- [ ] depends on: #26076
[](https://gitpod.io/from-referrer/)
|
t-algebraic-topology
merge-conflict
blocked-by-other-PR
WIP
|
1442/5 |
Mathlib.lean,Mathlib/AlgebraicTopology/SimplexCategory/Basic.lean,Mathlib/AlgebraicTopology/SimplicialSet/AnodyneExtensions/IsUniquelyCodimOneFace.lean,Mathlib/AlgebraicTopology/SimplicialSet/AnodyneExtensions/Pairing.lean,Mathlib/AlgebraicTopology/SimplicialSet/AnodyneExtensions/PairingCore.lean,Mathlib/AlgebraicTopology/SimplicialSet/AnodyneExtensions/Rank.lean,Mathlib/AlgebraicTopology/SimplicialSet/AnodyneExtensions/RankNat.lean,Mathlib/AlgebraicTopology/SimplicialSet/AnodyneExtensions/RelativeCellComplex.lean,Mathlib/AlgebraicTopology/SimplicialSet/Degenerate.lean,Mathlib/AlgebraicTopology/SimplicialSet/NonDegenerateSimplices.lean,Mathlib/AlgebraicTopology/SimplicialSet/NonDegenerateSimplicesSubcomplex.lean,Mathlib/AlgebraicTopology/SimplicialSet/Simplices.lean,Mathlib/AlgebraicTopology/SimplicialSet/StdSimplex.lean,Mathlib/CategoryTheory/EpiMono.lean,docs/references.bib |
15 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
12-3951 12 days ago |
25-83224 25 days ago |
0-1 1 second |
28351 |
joelriou author:joelriou |
feat(AlgebraicTopology/SimplicialSet): the rank function with values in natural numbers of a regular pairing |
Given a regular pairing `P` for a subcomplex of a simplicial, following the work by Sean Moss, *Another approach to the Kan-Quillen model structure*, we show that the rank function relative to the well founded ancestrality relation has values in the type of natural numbers.
---
- [ ] depends on: #28346
- [ ] depends on: #28336
- [ ] depends on: #28332
- [ ] depends on: #28330
- [ ] depends on: #28224
- [x] depends on: #27968
- [ ] depends on: #28034
- [ ] depends on: #26076
[](https://gitpod.io/from-referrer/)
|
t-algebraic-topology
merge-conflict
blocked-by-other-PR
WIP
|
1316/5 |
Mathlib.lean,Mathlib/AlgebraicTopology/SimplexCategory/Basic.lean,Mathlib/AlgebraicTopology/SimplicialSet/AnodyneExtensions/IsUniquelyCodimOneFace.lean,Mathlib/AlgebraicTopology/SimplicialSet/AnodyneExtensions/Pairing.lean,Mathlib/AlgebraicTopology/SimplicialSet/AnodyneExtensions/PairingCore.lean,Mathlib/AlgebraicTopology/SimplicialSet/AnodyneExtensions/Rank.lean,Mathlib/AlgebraicTopology/SimplicialSet/AnodyneExtensions/RankNat.lean,Mathlib/AlgebraicTopology/SimplicialSet/Degenerate.lean,Mathlib/AlgebraicTopology/SimplicialSet/NonDegenerateSimplices.lean,Mathlib/AlgebraicTopology/SimplicialSet/NonDegenerateSimplicesSubcomplex.lean,Mathlib/AlgebraicTopology/SimplicialSet/Simplices.lean,Mathlib/AlgebraicTopology/SimplicialSet/StdSimplex.lean,Mathlib/CategoryTheory/EpiMono.lean,docs/references.bib |
14 |
n/a |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
12-3946 12 days ago |
unknown |
unknown |
28346 |
joelriou author:joelriou |
feat(AlgebraicTopology/SimplicialSet): rank functions for pairings |
This PR introduces the type of (weak) rank functions for pairings, a notion introduced by Sean Moss, *Another approach to the Kan-Quillen model structure*. Rank functions can be used in order to show that certain pairings are regular (i.e. the ancestrality relation is well founded). In a future PR, it shall be shown that a regular pairing admits a rank function to the natural numbers, which shall be used to show that the corresponding inclusion of simplicial sets is a (strong) anodyne extension.
---
- [ ] depends on: #28336
- [ ] depends on: #28332
- [ ] depends on: #28330
- [ ] depends on: #28224
- [x] depends on: #27968
- [ ] depends on: #28034
- [ ] depends on: #26076
[](https://gitpod.io/from-referrer/)
|
t-algebraic-topology
merge-conflict
blocked-by-other-PR
WIP
|
1214/5 |
Mathlib.lean,Mathlib/AlgebraicTopology/SimplexCategory/Basic.lean,Mathlib/AlgebraicTopology/SimplicialSet/AnodyneExtensions/IsUniquelyCodimOneFace.lean,Mathlib/AlgebraicTopology/SimplicialSet/AnodyneExtensions/Pairing.lean,Mathlib/AlgebraicTopology/SimplicialSet/AnodyneExtensions/PairingCore.lean,Mathlib/AlgebraicTopology/SimplicialSet/AnodyneExtensions/Rank.lean,Mathlib/AlgebraicTopology/SimplicialSet/Degenerate.lean,Mathlib/AlgebraicTopology/SimplicialSet/NonDegenerateSimplices.lean,Mathlib/AlgebraicTopology/SimplicialSet/NonDegenerateSimplicesSubcomplex.lean,Mathlib/AlgebraicTopology/SimplicialSet/Simplices.lean,Mathlib/AlgebraicTopology/SimplicialSet/StdSimplex.lean,Mathlib/CategoryTheory/EpiMono.lean,docs/references.bib |
13 |
n/a |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
12-3944 12 days ago |
unknown |
unknown |
28336 |
joelriou author:joelriou |
feat(AlgebraicTopology/SimplicialSet): a helper structure to construct pairings |
In this PR, we introduce an helper structure `Subcomplex.PairingCore` in order to construct a pairing for a subcomplex of a simplicial set. The main differences with `Subcomplex.Pairing` are that we provide an index type `ι` in order to parametrize type (I) and type (II) simplices, and that the dimensions of these are definitionally `d` or `d + 1`.
---
- [ ] depends on: #28332
- [ ] depends on: #28330
- [ ] depends on: #28224
- [x] depends on: #27968
- [ ] depends on: #28034
- [ ] depends on: #26076
[](https://gitpod.io/from-referrer/)
|
t-algebraic-topology
merge-conflict
blocked-by-other-PR
WIP
|
1040/5 |
Mathlib.lean,Mathlib/AlgebraicTopology/SimplexCategory/Basic.lean,Mathlib/AlgebraicTopology/SimplicialSet/AnodyneExtensions/IsUniquelyCodimOneFace.lean,Mathlib/AlgebraicTopology/SimplicialSet/AnodyneExtensions/Pairing.lean,Mathlib/AlgebraicTopology/SimplicialSet/AnodyneExtensions/PairingCore.lean,Mathlib/AlgebraicTopology/SimplicialSet/Degenerate.lean,Mathlib/AlgebraicTopology/SimplicialSet/NonDegenerateSimplices.lean,Mathlib/AlgebraicTopology/SimplicialSet/NonDegenerateSimplicesSubcomplex.lean,Mathlib/AlgebraicTopology/SimplicialSet/Simplices.lean,Mathlib/AlgebraicTopology/SimplicialSet/StdSimplex.lean,Mathlib/CategoryTheory/EpiMono.lean,docs/references.bib |
12 |
4 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
12-3943 12 days ago |
25-83423 25 days ago |
0-2 2 seconds |
28332 |
joelriou author:joelriou |
feat(AlgebraicTopology/SimplicialSet): pairings of non degenerate simplices, following Sean Moss |
In this PR, we introduce the notion of pairing for a subcomplex of a simplicial set. Following the work of Sean Moss, *Another approach to the Kan-Quillen model structure*, this is an essential tool in the study of (inner) anodyne extensions.
---
- [ ] depends on: #28330
- [ ] depends on: #28224
- [x] depends on: #27968
- [ ] depends on: #28034
- [ ] depends on: #26076
[](https://gitpod.io/from-referrer/)
|
t-algebraic-topology
merge-conflict
blocked-by-other-PR
WIP
|
796/5 |
Mathlib.lean,Mathlib/AlgebraicTopology/SimplexCategory/Basic.lean,Mathlib/AlgebraicTopology/SimplicialSet/AnodyneExtensions/IsUniquelyCodimOneFace.lean,Mathlib/AlgebraicTopology/SimplicialSet/AnodyneExtensions/Pairing.lean,Mathlib/AlgebraicTopology/SimplicialSet/Degenerate.lean,Mathlib/AlgebraicTopology/SimplicialSet/NonDegenerateSimplices.lean,Mathlib/AlgebraicTopology/SimplicialSet/NonDegenerateSimplicesSubcomplex.lean,Mathlib/AlgebraicTopology/SimplicialSet/Simplices.lean,Mathlib/AlgebraicTopology/SimplicialSet/StdSimplex.lean,Mathlib/CategoryTheory/EpiMono.lean,docs/references.bib |
11 |
4 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
12-3942 12 days ago |
25-83426 25 days ago |
0-21 21 seconds |
28330 |
joelriou author:joelriou |
feat(AlgebraicTopology): the type of non degenerate simplices not in a given subcomplex |
---
- [ ] depends on: #28224
- [x] depends on: #27968
- [ ] depends on: #28034
- [ ] depends on: #26076
[](https://gitpod.io/from-referrer/)
|
t-algebraic-topology
merge-conflict
blocked-by-other-PR
WIP
|
576/5 |
Mathlib.lean,Mathlib/AlgebraicTopology/SimplexCategory/Basic.lean,Mathlib/AlgebraicTopology/SimplicialSet/Degenerate.lean,Mathlib/AlgebraicTopology/SimplicialSet/NonDegenerateSimplices.lean,Mathlib/AlgebraicTopology/SimplicialSet/NonDegenerateSimplicesSubcomplex.lean,Mathlib/AlgebraicTopology/SimplicialSet/Simplices.lean,Mathlib/AlgebraicTopology/SimplicialSet/StdSimplex.lean,Mathlib/CategoryTheory/EpiMono.lean |
8 |
4 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
12-3941 12 days ago |
25-83427 25 days ago |
0-2 2 seconds |
26291 |
RemyDegenne author:RemyDegenne |
feat(Probability): Fernique's theorem and Cameron-Martin theorem |
- invariance by rotation of Gaussian measures
- Fernique's theorem
- Corollary: the identity is in Lp for all finite p
- Definition of the Cameron-Martin space of a Gaussian measure
- The Cameron-Martin theorem: shifting a Gaussian measure by an element of the Cameron-Martin space gives an equivalent measure, and shifting by an element which is not in the Cameron-Martin space gives a mutually singular measure.
---
- [x] depends on: #24975
- [x] depends on: #24969
- [x] depends on: #24930
- [x] depends on: #24925
- [x] depends on: #24900
- [x] depends on: #25532
- [x] depends on: #27022
- [x] depends on: #27027
- [x] depends on: #27029
- [x] depends on: #27123
- [x] depends on: #27610
- [x] depends on: #28342
- [ ] depends on: #28343
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #24430.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/24430* |
t-measure-probability
blocked-by-other-PR
WIP
|
2664/5 |
Mathlib.lean,Mathlib/MeasureTheory/Measure/Portmanteau.lean,Mathlib/Probability/Distributions/Fernique.lean,Mathlib/Probability/Distributions/Gaussian/CameronMartin.lean,Mathlib/Probability/Distributions/Gaussian/CameronMartinThm.lean,Mathlib/Probability/Distributions/Gaussian/Fernique.lean,Mathlib/Probability/Distributions/Gaussian/Real.lean,Mathlib/Probability/Moments/CovarianceBilin.lean,Mathlib/Probability/Moments/Variance.lean,Mathlib/Topology/MetricSpace/ThickenedIndicator.lean,docs/1000.yaml,docs/references.bib |
12 |
6 |
['github-actions', 'grunweg', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
12-3573 12 days ago |
12-58471 12 days ago |
0-2 2 seconds |
25741 |
robin-carlier author:robin-carlier |
feat(AlgebraicTopology/SimplexCategory/SimplicialObject): definitions of simplicial objects by generators and relation |
We leverage the equivalence between `SimplexCategory` and `SimplexCategoryGenRel` to give new constructors for (co)simplicial objects, as well as constructors for natural transformations (resp. isomorphism) between those.
Final PR in the series of PR formalising the equivalence between `SimplexCategory` and `SimplexCategoryGenRel`.
---
- [ ] depends on: #25740
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #21748.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/21748* |
t-algebraic-topology
large-import
t-category-theory
merge-conflict
blocked-by-other-PR
|
1363/9 |
Mathlib.lean,Mathlib/AlgebraicTopology/SimplexCategory/GeneratorsRelations/Equivalence.lean,Mathlib/AlgebraicTopology/SimplexCategory/GeneratorsRelations/NormalForms.lean,Mathlib/AlgebraicTopology/SimplicialObject/GeneratorsRelations.lean |
4 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
12-584 12 days ago |
12-585 12 days ago |
11-15676 11 days |
25273 |
YaelDillies author:YaelDillies |
refactor: make `MonoidAlgebra` into a one-field structure |
From Toric
---
- [x] depends on: #26732
- [x] depends on: #28407
- [x] depends on: #28460
- [ ] depends on: #28511
- [ ] depends on: #29207
[](https://gitpod.io/from-referrer/)
|
toric
t-algebra
blocked-by-other-PR
WIP
label:t-algebra$ |
547/588 |
Mathlib/Algebra/BigOperators/Finsupp/Basic.lean,Mathlib/Algebra/Category/MonCat/Adjunctions.lean,Mathlib/Algebra/MonoidAlgebra/Defs.lean,Mathlib/Data/Finsupp/Multiset.lean,Mathlib/Data/Nat/Choose/Multinomial.lean,Mathlib/RepresentationTheory/Homological/GroupHomology/LowDegree.lean |
6 |
36 |
['JovanGerb', 'YaelDillies', 'alreadydone', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
11-77852 11 days ago |
12-79243 12 days ago |
36-61320 36 days |
28786 |
mitchell-horner author:mitchell-horner |
feat(Combinatorics/SimpleGraph): restate Turán's theorem in terms of `extremalNumber` |
Restates the existing proof of Turán's theorem in terms of the extremal numbers of `⊤`:
The `turanGraph` is, up to isomorphism, the unique extremal graph forbidding `⊤`.
---
- [ ] depends on: #28719
- [x] depends on: #28785
[](https://gitpod.io/from-referrer/)
|
t-combinatorics
blocked-by-other-PR
|
63/46 |
Mathlib/Combinatorics/SimpleGraph/Extremal/Turan.lean |
1 |
5 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
11-73200 11 days ago |
11-73220 11 days ago |
2-84097 2 days |
26104 |
xroblot author:xroblot |
feat(NumberField/IsCM): compute ratio of regulators |
This PR continues the work from #23696.
---
- [x] depends on: #23694
- [ ] depends on: #26075
- [ ] depends on: #26108 |
large-import
t-number-theory
merge-conflict
blocked-by-other-PR
|
681/85 |
Mathlib/Algebra/Field/Equiv.lean,Mathlib/Algebra/Group/Invertible/Basic.lean,Mathlib/Algebra/Module/ZLattice/Covolume.lean,Mathlib/AlgebraicGeometry/Morphisms/Proper.lean,Mathlib/FieldTheory/LinearDisjoint.lean,Mathlib/GroupTheory/GroupAction/FixedPoints.lean,Mathlib/GroupTheory/Index.lean,Mathlib/LinearAlgebra/Determinant.lean,Mathlib/LinearAlgebra/Dimension/Localization.lean,Mathlib/LinearAlgebra/Matrix/Determinant/Basic.lean,Mathlib/NumberTheory/NumberField/CMField.Lean,Mathlib/NumberTheory/NumberField/Units/Basic.lean,Mathlib/NumberTheory/NumberField/Units/DirichletTheorem.lean,Mathlib/NumberTheory/NumberField/Units/Regulator.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 |
21 |
4 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'xroblot'] |
nobody |
11-69440 11 days ago |
50-63035 1 month ago |
0-1395 23 minutes |
27707 |
FLDutchmann author:FLDutchmann |
feat(NumberTheory/SelbergSieve): define Selberg's weights and prove basic results. |
This PR continues the work from #23635.
Original PR: https://github.com/leanprover-community/mathlib4/pull/23635
- [ ] depends on: #27702 |
t-analysis
t-number-theory
merge-conflict
blocked-by-other-PR
|
407/83 |
Mathlib/NumberTheory/Divisors.lean,Mathlib/NumberTheory/SelbergSieve.lean |
2 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
11-53634 11 days ago |
11-53635 11 days ago |
3-375 3 days |
27898 |
grunweg author:grunweg |
feat: check indentation of doc-strings, basic version |
Basic version of #27897 (which still has some false positives): let's land this before weeding out the other errors.
---
- [x] depends on: #27895
- [x] depends on: #27901
- [ ] depends on: #27933
- a PR for adding clarifying newlines
- some miscellaneous indentation changes
[](https://gitpod.io/from-referrer/)
|
t-linter
merge-conflict
blocked-by-other-PR
|
510/268 |
Mathlib/Algebra/ContinuedFractions/Basic.lean,Mathlib/Algebra/Lie/Classical.lean,Mathlib/Algebra/Lie/OfAssociative.lean,Mathlib/Algebra/Module/LinearMap/Polynomial.lean,Mathlib/Algebra/Order/Hom/Basic.lean,Mathlib/Algebra/Polynomial/EraseLead.lean,Mathlib/Algebra/Polynomial/Inductions.lean,Mathlib/Algebra/Polynomial/Laurent.lean,Mathlib/CategoryTheory/Bicategory/NaturalTransformation/Oplax.lean,Mathlib/CategoryTheory/ConcreteCategory/Basic.lean,Mathlib/CategoryTheory/Enriched/Opposite.lean,Mathlib/CategoryTheory/Filtered/Basic.lean,Mathlib/CategoryTheory/Monoidal/Category.lean,Mathlib/CategoryTheory/Monoidal/Functor.lean,Mathlib/CategoryTheory/Monoidal/Limits/Basic.lean,Mathlib/CategoryTheory/NatIso.lean,Mathlib/CategoryTheory/Sites/Grothendieck.lean,Mathlib/CategoryTheory/Sites/Pretopology.lean,Mathlib/Combinatorics/Configuration.lean,Mathlib/Data/Bracket.lean,Mathlib/Data/Fin/Basic.lean,Mathlib/Data/Finsupp/MonomialOrder.lean,Mathlib/Data/Finsupp/MonomialOrder/DegLex.lean,Mathlib/Data/List/Defs.lean,Mathlib/Data/List/EditDistance/Defs.lean,Mathlib/Data/List/Rotate.lean,Mathlib/Data/Num/Basic.lean,Mathlib/Data/Num/Bitwise.lean,Mathlib/Data/Ordmap/Ordnode.lean,Mathlib/Data/PNat/Xgcd.lean,Mathlib/Data/Part.lean,Mathlib/Geometry/Manifold/LocalDiffeomorph.lean,Mathlib/Geometry/RingedSpace/PresheafedSpace/Gluing.lean,Mathlib/GroupTheory/GroupAction/MultiplePrimitivity.lean,Mathlib/MeasureTheory/Function/AEEqOfIntegral.lean,Mathlib/MeasureTheory/Group/Action.lean,Mathlib/NumberTheory/FLT/Basic.lean,Mathlib/NumberTheory/RamificationInertia/Basic.lean,Mathlib/Order/Filter/Partial.lean,Mathlib/Order/Interval/Finset/Defs.lean,Mathlib/RingTheory/DividedPowers/Basic.lean,Mathlib/Tactic/Bound/Attribute.lean,Mathlib/Tactic/ComputeDegree.lean,Mathlib/Tactic/Linter/DocString.lean,Mathlib/Tactic/MinImports.lean,Mathlib/Tactic/MoveAdd.lean,Mathlib/Tactic/RewriteSearch.lean,Mathlib/Tactic/Sat/FromLRAT.lean,Mathlib/Tactic/TermCongr.lean,Mathlib/Tactic/ToAdditive/Frontend.lean,Mathlib/Util/Notation3.lean,Mathlib/Util/Superscript.lean,MathlibTest/DocString.lean,MathlibTest/slow_simp.lean |
54 |
6 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
11-53633 11 days ago |
11-53634 11 days ago |
0-26 26 seconds |
29164 |
vlad902 author:vlad902 |
feat(SimpleGraph): Hall's Marriage Theorem for bipartite graphs |
Derive the graph theoretic proof of Hall's marriage theorem from the combinatorial version.
Note that I specifically implement this for the more general case of infinite graphs that are locally finite (e.g. every vertex has only finite neighbors.) As a result, the theorem depends on some category theoretic infrastructure required for the infinite combinatorial formulation of Hall's Marriage Theorem and hence I've placed the theorems into their own file to avoid requiring it in `Matching.lean`
- [ ] depends on: #29162 |
t-combinatorics
blocked-by-other-PR
|
133/7 |
Mathlib/Combinatorics/Hall/Basic.lean,Mathlib/Combinatorics/SimpleGraph/Hall.lean,Mathlib/Combinatorics/SimpleGraph/Matching.lean,docs/1000.yaml |
4 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
10-59668 10 days ago |
11-5614 11 days ago |
0-3248 54 minutes |
28126 |
Sebi-Kumar author:Sebi-Kumar |
feat(AlgebraicTopology/FundamentalGroupoid): relate equality in fundamental groupoid to homotopy |
Prove the theorem `fromPath_eq_iff_homotopic` which shows that two paths are equal in the fundamental groupoid if and only if they are homotopic. Also add simp lemmas `fromPath_refl`, `fromPath_symm`, and `fromPath_trans`. Together, these allow one to prove two paths are homotopic by transferring to the fundamental groupoid and using the `aesop_cat` tactic.
---
I would like to thank Kenny Lau for inspiring this code on Zulip at [#Is there code for X? > Using aesop_cat to prove paths are homotopic](https://leanprover.zulipchat.com/#narrow/channel/217875-Is-there-code-for-X.3F/topic/Using.20aesop_cat.20to.20prove.20paths.20are.20homotopic).
Also, I would like to note that I am a newcomer when it comes to contributing to Mathlib, and that this code was written as a part of a formalization project at the University of Western Ontario under the supervision of Chris Kapulkin and Daniel Carranza (which is happening through the Fields Undergraduate Summer Research Program).
- [ ] depends on: #28234
[](https://gitpod.io/from-referrer/)
|
t-algebraic-topology
new-contributor
awaiting-author
blocked-by-other-PR
|
121/141 |
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/Product.lean |
8 |
10 |
['Sebi-Kumar', 'alreadydone', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'mattrobball'] |
mattrobball assignee:mattrobball |
10-56272 10 days ago |
10-56272 10 days ago |
14-30316 14 days |
28017 |
eric-wieser author:eric-wieser |
feat: generalize some opnorm lemmas to seminormed spaces |
---
- [ ] depends on: #28014
- [ ] depends on: #28101
- [ ] depends on: #29120
[](https://gitpod.io/from-referrer/)
|
t-analysis
merge-conflict
blocked-by-other-PR
WIP
|
60/24 |
Mathlib/Analysis/NormedSpace/OperatorNorm/NNNorm.lean,Mathlib/Analysis/NormedSpace/Real.lean |
2 |
5 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
10-39116 10 days ago |
10-39117 10 days ago |
0-0 0 seconds |
27675 |
EtienneC30 author:EtienneC30 |
feat: introduce `covInnerBilin` |
`covInnerBilin` is the covariance bilinear form associated with a measure on an inner product space.
from BrownianMotion
---
- [ ] depends on: #27626
- [x] depends on: #27674
Co-authored-by: Rémy Degenne @RemyDegenne
[](https://gitpod.io/from-referrer/)
|
large-import
t-measure-probability
merge-conflict
blocked-by-other-PR
|
695/2 |
Mathlib.lean,Mathlib/Analysis/NormedSpace/ContinuousBilinForm.lean,Mathlib/LinearAlgebra/BilinearForm/IsPosSemidef.lean,Mathlib/LinearAlgebra/Matrix/BilinearForm.lean,Mathlib/LinearAlgebra/Matrix/Hermitian.lean,Mathlib/MeasureTheory/Integral/Eval/Basic.lean,Mathlib/MeasureTheory/Integral/Eval/WithLp.lean,Mathlib/Probability/Moments/CovInnerBilin.lean,Mathlib/Probability/Moments/CovarianceBilin.lean |
9 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
10-18460 10 days ago |
32-21437 1 month ago |
0-1309 21 minutes |
29283 |
Jlh18 author:Jlh18 |
feat(CategoryTheory): define forgetful-core adjunction between Cat and Grpd |
* Define `CategoryTheory.Core.functor`: the functor `Cat ⥤ Grpd` that on objects takes
the core of a category
* Define `CategoryTheory.Core.adjunction`: the adjunction with the forgetful functor
`Grpd.forgetToCat` on the left, and the core functor `Core.functor` on the right.
* Hence provide an instance that `Grpd.forgetToCat` is coreflective.
- [ ] depends on: #29284 [Extra lemmas in CategoryTheory.Core]
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
blocked-by-other-PR
|
104/4 |
Mathlib.lean,Mathlib/AlgebraicTopology/FundamentalGroupoid/InducedMaps.lean,Mathlib/CategoryTheory/Category/Grpd.lean,Mathlib/CategoryTheory/Core.lean,Mathlib/CategoryTheory/Groupoid/Grpd/Core.lean |
5 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
9-76946 9 days ago |
10-26365 10 days ago |
0-3572 59 minutes |
29282 |
Jlh18 author:Jlh18 |
feat(CategoryTheory): HasColimits instance onGrpd |
Show that the category of groupoids has all small colimits, as a coreflective subcategory of `Cat`, which has all small colimits. The right adjoint of the forgetful functor is the core functor `CategoryTheory.Core.functor`.
- [ ] depends on: #29283 [Core of a category as a functor]
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
blocked-by-other-PR
|
140/4 |
Mathlib.lean,Mathlib/AlgebraicTopology/FundamentalGroupoid/InducedMaps.lean,Mathlib/CategoryTheory/Category/Grpd.lean,Mathlib/CategoryTheory/Core.lean,Mathlib/CategoryTheory/Groupoid/Grpd/Colimit.lean,Mathlib/CategoryTheory/Groupoid/Grpd/Core.lean |
6 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
9-76879 9 days ago |
10-29794 10 days ago |
0-396 6 minutes |
29284 |
Jlh18 author:Jlh18 |
feat(CategoryTheory): naturality lemmas for Core construction |
Lemmas for PR #29283 to prove that `Core` is the right adjoint to the forgetful functor from `Cat` to `Grpd`.
These lemmas are more general than that setting, and need not be stated in the bundled format.
- [ ] depends on: #29250
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
blocked-by-other-PR
|
35/4 |
Mathlib/AlgebraicTopology/FundamentalGroupoid/InducedMaps.lean,Mathlib/CategoryTheory/Category/Grpd.lean,Mathlib/CategoryTheory/Core.lean |
3 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
9-76857 9 days ago |
9-78158 9 days ago |
0-37819 10 hours |
25841 |
mitchell-horner author:mitchell-horner |
feat(Combinatorics/SimpleGraph): prove the Kővári–Sós–Turán theorem |
Prove the Kővári–Sós–Turán theorem for simple graphs:
The `(completeBipartiteGraph α β).Free` simple graphs for `card α ≤ card β` on the vertex type `V` have at most `(card β-1)^(1/(card α))*(card V)^(2-1/(card α))/2 + (card V)*(card α-1)/2` edges.
The double-counting construction from the proof is available in `namespace KovariSosTuran`.
---
- [x] depends on: #19865
- [x] depends on: #20738
- [ ] depends on: #27602
I've tried to make as much of the double-counting construction not private as possible. I figure it is useful to borrow constructions between proofs.
If this is just considered garbage and bloat and better left private. Please let me know.
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #20240.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/20240* |
t-combinatorics
blocked-by-other-PR
WIP
|
283/0 |
Mathlib.lean,Mathlib/Combinatorics/SimpleGraph/Bipartite.lean,Mathlib/Combinatorics/SimpleGraph/Extremal/KovariSosTuran.lean |
3 |
4 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
9-69307 9 days ago |
9-70715 9 days ago |
45-15427 45 days |
27706 |
xroblot author:xroblot |
feat(RingTheory/Localization/AtPrime): inertia degree and ramification index are preserved by localization |
Let `R ⊆ S` be an extension of rings and `p` be a prime ideal of `R`. Denote by `Rₚ` the localization of `R` at the complement of `p` and by `Sₚ` the localization of `S` at the (image) of the complement of `p`.
In this PR, we prove that the bijection between the (nonzero) prime ideals of `Sₚ` and the prime ideals of `S` above `p` preserves the residual degree and the ramification index.
---
- [x] depends on: #27794
- [x] depends on: #27796
- [x] depends on: #27798
- [x] depends on: #28526
- [ ] depends on: #29322
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
blocked-by-other-PR
WIP
|
508/122 |
Mathlib.lean,Mathlib/NumberTheory/RamificationInertia/Basic.lean,Mathlib/RingTheory/DedekindDomain/Instances.lean,Mathlib/RingTheory/Ideal/Maps.lean,Mathlib/RingTheory/Ideal/Over.lean,Mathlib/RingTheory/Localization/AtPrime/Basic.lean,Mathlib/RingTheory/Localization/AtPrime/Extension.lean,Mathlib/RingTheory/Trace/Quotient.lean |
8 |
4 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
9-9670 9 days ago |
9-65926 9 days ago |
0-1400 23 minutes |
27970 |
smmercuri author:smmercuri |
feat: collections of distinct infinite places contain values that diverge around 1 |
This PR continues the work from #22147.
Original PR: https://github.com/leanprover-community/mathlib4/pull/22147
---
- [ ] depends on: #27969 |
large-import
t-algebra
t-number-theory
merge-conflict
blocked-by-other-PR
label:t-algebra$ |
1647/1 |
Mathlib/Algebra/Order/AbsoluteValue/Basic.lean,Mathlib/Analysis/AbsoluteValue/Equivalence.lean,Mathlib/Analysis/Normed/Ring/WithAbs.lean,Mathlib/Data/Fin/Basic.lean,Mathlib/Data/Finset/Lattice/Fold.lean,Mathlib/Logic/Pairwise.lean,Mathlib/NumberTheory/NumberField/Embeddings.lean |
7 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
9-7420 9 days ago |
9-7421 9 days ago |
0-2827 47 minutes |
28972 |
themathqueen author:themathqueen |
feat(LinearAlgebra/Matrix): star-algebra automorphisms on matrices are unitarily inner |
Characterization of star-algebra automorphisms on matrices: for any star-algebra automorphism `f` on matrices, there exists a unitary matrix `U` such that `f x = U * x * star U`.
---
- [ ] depends on: #28100
- [x] depends on: #28182
- [x] depends on: #28881
[](https://gitpod.io/from-referrer/)
|
t-algebra
blocked-by-other-PR
label:t-algebra$ |
155/0 |
Mathlib.lean,Mathlib/LinearAlgebra/Matrix/GeneralLinearGroup/Basic.lean,Mathlib/LinearAlgebra/Matrix/StarAlgEquiv.lean |
3 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
8-79054 8 days ago |
17-68033 17 days ago |
0-412 6 minutes |
27668 |
IvanRenison author:IvanRenison |
feat(Analysis/InnerProductSpace): define outer product of linear maps |
Co-authored-by: Jam Kabeer Ali Khan
---
I'm not completely sure if this is a good addition or not, and also, I was not sure if to call the definition `outerProduct` or only `outer`.
- [ ] depends on: #28350
- [ ] depends on: #28344
[](https://gitpod.io/from-referrer/)
|
t-analysis
blocked-by-other-PR
|
205/8 |
Mathlib.lean,Mathlib/Algebra/Module/LinearMap/Lemmas.lean,Mathlib/Analysis/InnerProductSpace/Adjoint.lean,Mathlib/Analysis/InnerProductSpace/Dual.lean,Mathlib/Analysis/InnerProductSpace/LinearMap.lean,Mathlib/Analysis/InnerProductSpace/PiL2.lean,Mathlib/Analysis/InnerProductSpace/Positive.lean,Mathlib/Analysis/InnerProductSpace/Trace.lean,Mathlib/LinearAlgebra/Dual/Lemmas.lean,Mathlib/Topology/Algebra/Module/LinearMap.lean |
10 |
69 |
['IvanRenison', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'themathqueen'] |
themathqueen assignee:themathqueen |
8-76937 8 days ago |
8-78055 8 days ago |
2-50264 2 days |
27314 |
pechersky author:pechersky |
feat(TopologyValued): `Valued` based on a range topology |
Switch from a topology based on `fun γ : Γ₀ˣ => (v.ltAddSubgroup γ : AddSubgroup R)` to
```
fun rs : {rs : R × R // v rs.1 ≠ 0 ∧ v rs.2 ≠ 0} ↦
(v.ltAddSubgroup (Units.mk0 (v rs.val.2 / v rs.val.1) (by simp [rs.prop])) : AddSubgroup R)
```
This is in preparation for using `IsValuativeTopology` instead. In fact, that basis is precisely what `ValuativeTopology` asserts.
`Valued.mk'` is kept, we do not yet rely on `IsValuativeTopology` and `UniformSpace`.
The new `Valued` behaves the same way as it did before for `MulArchimedean` valuation codomains, which are all of the current in-mathlib uses of `Valued`. This is, for rank-one valuations. For valuations which rank one, but do not pass to the whole codomain, there are helper lemmas to discuss open/closed/clopen sets.
---
[](https://gitpod.io/from-referrer/)
- [x] depends on: #27264
- [x] depends on: #27265
- [ ] depends on: #27163
- [ ] depends on: #27339 |
t-topology
merge-conflict
blocked-by-other-PR
|
733/259 |
Mathlib/Analysis/Normed/Field/Basic.lean,Mathlib/FieldTheory/RatFunc/AsPolynomial.lean,Mathlib/NumberTheory/FunctionField.lean,Mathlib/RingTheory/LaurentSeries.lean,Mathlib/RingTheory/Valuation/ValuativeRel.lean,Mathlib/Topology/Algebra/Valued/LocallyCompact.lean,Mathlib/Topology/Algebra/Valued/NormedValued.lean,Mathlib/Topology/Algebra/Valued/ValuationTopology.lean,Mathlib/Topology/Algebra/Valued/ValuativeRel.lean,Mathlib/Topology/Algebra/Valued/ValuedField.lean,Mathlib/Topology/Algebra/Valued/WithVal.lean,Mathlib/Topology/Algebra/Valued/WithZeroMulInt.lean |
12 |
9 |
['github-actions', 'kckennylau', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
8-69457 8 days ago |
33-66794 1 month ago |
0-22127 6 hours |
29336 |
bryangingechen author:bryangingechen |
testing for #27956: remove deprecations older than 2025-02-28 |
These were the changes made by running `python3 scripts/remove_deprecated_decls.py 2025-02-28` on 8d55c35c2683b1ce9656b33035ef1392b563ca09.
---
- [ ] depends on: #27956
[](https://gitpod.io/from-referrer/)
|
test-ci
merge-conflict
blocked-by-other-PR
|
330/1168 |
.github/workflows/remove_deprecated_decls.yml,Mathlib/Combinatorics/Matroid/Circuit.lean,Mathlib/Combinatorics/Matroid/Closure.lean,Mathlib/Combinatorics/Matroid/Minor/Restrict.lean,Mathlib/Computability/Halting.lean,Mathlib/Computability/Partrec.lean,Mathlib/Computability/Primrec.lean,Mathlib/Data/ENNReal/Basic.lean,Mathlib/Data/Fin/Basic.lean,Mathlib/Data/Fin/SuccPred.lean,Mathlib/Data/Finite/Card.lean,Mathlib/Data/Finset/Basic.lean,Mathlib/Data/Fintype/BigOperators.lean,Mathlib/Data/List/Basic.lean,Mathlib/Data/List/Cycle.lean,Mathlib/Data/List/GetD.lean,Mathlib/Data/List/MinMax.lean,Mathlib/Data/List/ModifyLast.lean,Mathlib/Data/List/Nodup.lean,Mathlib/Data/List/NodupEquivFin.lean,Mathlib/Data/List/OfFn.lean,Mathlib/Data/List/ReduceOption.lean,Mathlib/Data/List/Rotate.lean,Mathlib/Data/List/Scan.lean,Mathlib/Data/List/TakeDrop.lean,Mathlib/Data/List/Zip.lean,Mathlib/Data/Matrix/ColumnRowPartitioned.lean,Mathlib/Data/Multiset/Basic.lean,Mathlib/Data/Seq/Defs.lean,Mathlib/Data/Set/Finite/Basic.lean,Mathlib/Data/Set/List.lean,Mathlib/Data/Set/Operations.lean,Mathlib/Data/Set/Prod.lean,Mathlib/Data/Stream/Init.lean,Mathlib/Data/String/Lemmas.lean,Mathlib/Data/Sum/Basic.lean,Mathlib/Geometry/Manifold/ContMDiff/Constructions.lean,Mathlib/Geometry/RingedSpace/Basic.lean,Mathlib/GroupTheory/GroupAction/SubMulAction.lean,Mathlib/GroupTheory/Perm/Cycle/Concrete.lean,Mathlib/LinearAlgebra/AffineSpace/AffineSubspace/Basic.lean,Mathlib/LinearAlgebra/Dimension/Constructions.lean,Mathlib/LinearAlgebra/Dimension/RankNullity.lean,Mathlib/LinearAlgebra/LinearIndependent/Basic.lean,Mathlib/LinearAlgebra/LinearIndependent/Defs.lean,Mathlib/LinearAlgebra/LinearIndependent/Lemmas.lean,Mathlib/Logic/Equiv/Basic.lean,Mathlib/Logic/Equiv/List.lean,Mathlib/MeasureTheory/Function/ConditionalExpectation/AEMeasurable.lean,Mathlib/MeasureTheory/Function/ConditionalExpectation/Basic.lean,Mathlib/MeasureTheory/Function/ContinuousMapDense.lean,Mathlib/MeasureTheory/Function/L1Space/Integrable.lean,Mathlib/MeasureTheory/Function/L2Space.lean,Mathlib/MeasureTheory/Function/LocallyIntegrable.lean,Mathlib/MeasureTheory/Function/LpOrder.lean,Mathlib/MeasureTheory/Function/LpSeminorm/ChebyshevMarkov.lean,Mathlib/MeasureTheory/Function/LpSeminorm/CompareExp.lean,Mathlib/MeasureTheory/Function/LpSeminorm/Defs.lean,Mathlib/MeasureTheory/Function/LpSeminorm/Trim.lean,Mathlib/MeasureTheory/Function/LpSpace/Basic.lean,Mathlib/MeasureTheory/Function/LpSpace/Complete.lean,Mathlib/MeasureTheory/Function/LpSpace/Indicator.lean,Mathlib/MeasureTheory/Function/StronglyMeasurable/Lp.lean,Mathlib/MeasureTheory/Integral/Bochner/Basic.lean,Mathlib/MeasureTheory/Integral/CircleTransform.lean,Mathlib/MeasureTheory/Integral/IntegrableOn.lean,Mathlib/MeasureTheory/Integral/Lebesgue/Countable.lean,Mathlib/MeasureTheory/Measure/Content.lean,Mathlib/MeasureTheory/Measure/Count.lean,Mathlib/ModelTheory/Basic.lean,Mathlib/ModelTheory/Definability.lean,Mathlib/ModelTheory/ElementarySubstructures.lean,Mathlib/ModelTheory/LanguageMap.lean,Mathlib/ModelTheory/Semantics.lean,Mathlib/ModelTheory/Substructures.lean,Mathlib/ModelTheory/Syntax.lean,Mathlib/NumberTheory/Divisors.lean,Mathlib/NumberTheory/ModularForms/EisensteinSeries/IsBoundedAtImInfty.lean,Mathlib/NumberTheory/NumberField/House.lean,Mathlib/Order/Filter/AtTopBot/Monoid.lean,Mathlib/Order/Filter/AtTopBot/Ring.lean,Mathlib/Order/GaloisConnection/Basic.lean,Mathlib/Order/Max.lean,Mathlib/Order/WithBot.lean,Mathlib/Probability/IdentDistrib.lean,Mathlib/Probability/Independence/Integrable.lean,Mathlib/Probability/Martingale/Convergence.lean,Mathlib/Probability/Moments/ComplexMGF.lean,Mathlib/Probability/Moments/IntegrableExpMul.lean,Mathlib/Probability/Moments/Variance.lean,Mathlib/Probability/Process/Filtration.lean,Mathlib/RingTheory/Algebraic/Integral.lean,Mathlib/RingTheory/AlgebraicIndependent/AlgebraicClosure.lean,Mathlib/RingTheory/AlgebraicIndependent/Basic.lean,Mathlib/RingTheory/Ideal/Maps.lean,Mathlib/RingTheory/NonUnitalSubsemiring/Defs.lean,Mathlib/RingTheory/Spectrum/Prime/Topology.lean,Mathlib/SetTheory/Ordinal/Arithmetic.lean,Mathlib/SetTheory/Ordinal/Basic.lean,Mathlib/SetTheory/Ordinal/Family.lean |
119 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
8-62815 8 days ago |
9-6727 9 days ago |
0-0 0 seconds |
29357 |
eric-wieser author:eric-wieser |
refactor: generalize IsSimpleRing to semirings |
---
- [ ] depends on: #26277
- [ ] depends on: #22954
[](https://gitpod.io/from-referrer/)
|
blocked-by-other-PR |
26/9 |
Mathlib/Data/Setoid/Basic.lean,Mathlib/RingTheory/SimpleRing/Basic.lean,Mathlib/RingTheory/SimpleRing/Defs.lean |
3 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
8-426 8 days ago |
8-428 8 days ago |
0-0 0 seconds |
29258 |
mans0954 author:mans0954 |
feature(Analysis/LocallyConvex/WeakSpace): weak closed convex hull equals closed convex hull |
The weak closed convex hull is equal to the closed convex hull in the original topology.
---
- [ ] depends on: #29248
[](https://gitpod.io/from-referrer/)
|
t-analysis
blocked-by-other-PR
|
59/0 |
Mathlib/Analysis/Convex/Basic.lean,Mathlib/Analysis/LocallyConvex/WeakSpace.lean,Mathlib/Analysis/RCLike/Lemmas.lean |
3 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
6-10420 6 days ago |
7-2927 7 days ago |
0-2635 43 minutes |
29342 |
mans0954 author:mans0954 |
refactor(Analysis/LocallyConvex/AbsConvex): Redefine AbsConvex to use a single ring of scalars |
Currently the definition of Absolutely Convex in Mathlib is a little unexpected:
```
def AbsConvex (s : Set E) : Prop := Balanced 𝕜 s ∧ Convex ℝ s
```
At the time this definition was formulated, Mathlib's definition of `Convex` required the scalars to be an `OrderedSemiring` whereas the definition of `Balanced` required the scalars to be a `SeminormedRing`. Mathlib didn't have a concept of a semi-normed ordered ring, so a set was defined as `AbsConvex` if it is balanced over a `SeminormedRing` `𝕜` and convex over `ℝ`.
Recently the requirements for the definition of `Convex` have been relaxed (#24392, #20595) so it is now possible to use a single scalar ring in common with the liturature.
Previous discussion:
- https://github.com/leanprover-community/mathlib4/pull/17029#discussion_r1782249323
- https://github.com/leanprover-community/mathlib4/pull/26345#discussion_r2287535746
---
- [ ] depends on: #29248
[](https://gitpod.io/from-referrer/)
|
t-analysis
blocked-by-other-PR
|
106/68 |
Mathlib/Analysis/Convex/Basic.lean,Mathlib/Analysis/LocallyConvex/AbsConvex.lean,Mathlib/Analysis/LocallyConvex/AbsConvexOpen.lean,Mathlib/Analysis/LocallyConvex/Basic.lean,Mathlib/Analysis/Normed/Module/Dual.lean,Mathlib/Analysis/RCLike/Lemmas.lean |
6 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
6-9600 6 days ago |
7-4994 7 days ago |
0-12 12 seconds |
29343 |
themathqueen author:themathqueen |
feat(LinearAlgebra/TensorProduct/Basic): add `range_map_mono` |
---
- [ ] depends on: #29391
[](https://gitpod.io/from-referrer/)
|
t-algebra
blocked-by-other-PR
label:t-algebra$ |
56/12 |
Mathlib/Algebra/Lie/TensorProduct.lean,Mathlib/Algebra/Module/Submodule/Bilinear.lean,Mathlib/LinearAlgebra/TensorProduct/Basic.lean,Mathlib/LinearAlgebra/TensorProduct/Quotient.lean |
4 |
4 |
['eric-wieser', 'github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
5-86158 5 days ago |
5-86180 5 days ago |
2-82385 2 days |
29378 |
mans0954 author:mans0954 |
feature(Analysis/LocallyConvex/AbsConvex): Balanced and AbsConvex sets under linear maps |
Provide `Balanced` and `AbsConvex` versions of `Convex.linear_image`, `Convex.linear_preimage` and the `is_linear` equivalents.
---
- [ ] depends on: #29342
[](https://gitpod.io/from-referrer/)
|
t-analysis
blocked-by-other-PR
|
184/68 |
Mathlib/Analysis/Convex/Basic.lean,Mathlib/Analysis/LocallyConvex/AbsConvex.lean,Mathlib/Analysis/LocallyConvex/AbsConvexOpen.lean,Mathlib/Analysis/LocallyConvex/BalancedCoreHull.lean,Mathlib/Analysis/LocallyConvex/Basic.lean,Mathlib/Analysis/Normed/Module/Dual.lean,Mathlib/Analysis/RCLike/Lemmas.lean |
7 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
5-83747 5 days ago |
6-84228 6 days ago |
0-424 7 minutes |
29393 |
staroperator author:staroperator |
feat(SetTheory/ZFC): `card (V_ o) = preBeth o` |
---
- [ ] depends on: #26544
- [ ] depends on: #29351
- [ ] depends on: #29365
[](https://gitpod.io/from-referrer/)
|
blocked-by-other-PR |
231/41 |
Mathlib.lean,Mathlib/Data/W/Cardinal.lean,Mathlib/ModelTheory/Encoding.lean,Mathlib/SetTheory/Cardinal/Arithmetic.lean,Mathlib/SetTheory/Cardinal/Basic.lean,Mathlib/SetTheory/Cardinal/Cofinality.lean,Mathlib/SetTheory/Cardinal/Defs.lean,Mathlib/SetTheory/Cardinal/Order.lean,Mathlib/SetTheory/Cardinal/Ordinal.lean,Mathlib/SetTheory/Cardinal/Pigeonhole.lean,Mathlib/SetTheory/Cardinal/Regular.lean,Mathlib/SetTheory/ZFC/Basic.lean,Mathlib/SetTheory/ZFC/Cardinal.lean,Mathlib/SetTheory/ZFC/VonNeumann.lean |
14 |
4 |
['github-actions', 'mathlib4-dependent-issues-bot', 'staroperator', 'vihdzp'] |
nobody |
5-77066 5 days ago |
6-31885 6 days ago |
0-0 0 seconds |
29387 |
mans0954 author:mans0954 |
feature(Analysis/LocallyConvex/WeakSpace): toWeakSpace_closedAbsConvexHull_eq |
The closed absolutely convex hull taken in the weak topology coincides with the closed absolutely convex hull taken in the original topology.
---
- [ ] depends on: #29378
[](https://gitpod.io/from-referrer/)
|
t-analysis
blocked-by-other-PR
|
196/68 |
Mathlib/Analysis/Convex/Basic.lean,Mathlib/Analysis/LocallyConvex/AbsConvex.lean,Mathlib/Analysis/LocallyConvex/AbsConvexOpen.lean,Mathlib/Analysis/LocallyConvex/BalancedCoreHull.lean,Mathlib/Analysis/LocallyConvex/Basic.lean,Mathlib/Analysis/LocallyConvex/WeakSpace.lean,Mathlib/Analysis/Normed/Module/Dual.lean,Mathlib/Analysis/RCLike/Lemmas.lean |
8 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
5-75272 5 days ago |
6-58029 6 days ago |
0-2474 41 minutes |
26942 |
pechersky author:pechersky |
feat(RingTheory/Valuation/ValueGroupIso): isomorphism of value groups when compatible |
and also to the ValuativeRel's value group
by request from comment in
https://github.com/leanprover-community/mathlib4/pull/26754#issuecomment-3051770901
- [ ] depends on: #26588
---
[](https://gitpod.io/from-referrer/)
- [x] depends on: #26939
- [x] depends on: #26940
- [x] depends on: #26941 |
t-ring-theory
t-order
blocked-by-other-PR
|
235/0 |
Mathlib.lean,Mathlib/Algebra/GroupWithZero/Range.lean,Mathlib/Algebra/Order/GroupWithZero/Range.lean,Mathlib/Algebra/Order/Monoid/WithTop.lean,Mathlib/RingTheory/Valuation/ValueGroupIso.lean |
5 |
8 |
['faenuccio', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'pechersky'] |
faenuccio assignee:faenuccio |
5-29933 5 days ago |
5-62576 5 days ago |
10-67838 10 days |
29425 |
pechersky author:pechersky |
feat(NumberTheory/Padics/Torsion): `HasEnoughRootsOfUnity ℤ_[p] (p - 1)` |
---
[](https://gitpod.io/from-referrer/)
- [ ] depends on: #29403
- [ ] depends on: #29404
- [ ] depends on: #29405
- [ ] depends on: #29408
- [ ] depends on: #29424
|
t-ring-theory
blocked-by-other-PR
|
383/0 |
Mathlib.lean,Mathlib/Analysis/Normed/Group/Ultra.lean,Mathlib/Data/Nat/Basic.lean,Mathlib/Data/Nat/Choose/Dvd.lean,Mathlib/Data/Nat/Prime/Factorial.lean,Mathlib/NumberTheory/Padics/PadicIntegers.lean,Mathlib/NumberTheory/Padics/PadicNumbers.lean,Mathlib/NumberTheory/Padics/RingHoms.lean,Mathlib/NumberTheory/Padics/Torsion.lean,Mathlib/RingTheory/RootsOfUnity/EnoughRootsOfUnity.lean,Mathlib/RingTheory/ZMod/Torsion.lean |
11 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
5-29526 5 days ago |
5-29527 5 days ago |
0-657 10 minutes |
29424 |
pechersky author:pechersky |
feat(RingTheory/ZMod): `HasEnoughRootsOfUnity (ZMod p) (p - 1)` |
---
[](https://gitpod.io/from-referrer/)
- [ ] depends on: #29416
Not sure if this belongs better in `UnitsCyclic.lean` |
t-ring-theory
blocked-by-other-PR
|
47/0 |
Mathlib.lean,Mathlib/RingTheory/RootsOfUnity/EnoughRootsOfUnity.lean,Mathlib/RingTheory/ZMod/Torsion.lean |
3 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
5-29525 5 days ago |
5-29525 5 days ago |
0-2247 37 minutes |
29418 |
jsm28 author:jsm28 |
feat(Analysis/Convex/Between): interior of a 1-simplex |
Add lemmas relating the `interior` or `closedInterior` of a 1-simplex to betweenness.
---
- [ ] depends on: #29415
- [ ] depends on: #29422
[](https://gitpod.io/from-referrer/)
|
t-convex-geometry
blocked-by-other-PR
|
113/4 |
Mathlib/Analysis/Convex/Between.lean,Mathlib/Data/Finset/Max.lean |
2 |
6 |
['eric-wieser', 'github-actions', 'jsm28', 'mathlib4-dependent-issues-bot'] |
nobody |
5-1772 5 days ago |
5-36280 5 days ago |
0-328 5 minutes |
29415 |
jsm28 author:jsm28 |
feat(Data/Finset/Max): `min'_pair`, `max'_pair` |
Add the lemmas:
```lean
@[simp] lemma min'_pair (a b : α) : min' {a, b} (insert_nonempty _ _) = min a b := by
```
```lean
@[simp] lemma max'_pair (a b : α) : max' {a, b} (insert_nonempty _ _) = max a b := by
```
---
- [ ] depends on: #29422
[](https://gitpod.io/from-referrer/)
|
t-data
blocked-by-other-PR
|
20/4 |
Mathlib/Data/Finset/Max.lean |
1 |
11 |
['eric-wieser', 'github-actions', 'jsm28', 'mathlib4-dependent-issues-bot'] |
nobody |
5-1711 5 days ago |
5-1711 5 days ago |
0-5565 1 hour |
28895 |
yury-harmonic author:yury-harmonic |
feat(NumberTheory): prove Zsigmondy's theorem |
---
- [x] depends on: #28879
- [x] depends on: #28825
- [ ] depends on: #28833
- [x] depends on: #28888
- [x] depends on: #28830
- [x] depends on: #28765
- [x] depends on: #28886
- [ ] depends on: #28934
[](https://gitpod.io/from-referrer/)
|
blocked-by-other-PR |
1467/18 |
Mathlib.lean,Mathlib/Algebra/MvPolynomial/Eval.lean,Mathlib/Algebra/MvPolynomial/Expand.lean,Mathlib/NumberTheory/Zsigmondy.lean,Mathlib/Tactic.lean,Mathlib/Tactic/NormNum/Parity.lean,scripts/noshake.json |
7 |
7 |
['dupuisf', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'yury-harmonic'] |
nobody |
4-67671 4 days ago |
15-3656 15 days ago |
0-0 0 seconds |
26304 |
Raph-DG author:Raph-DG |
feat(AlgebraicGeometry): Definition of algebraic cycles |
In this PR we define algebraic cycles on a scheme X to be functions from the points of X to the integers with locally finite support. We introduce some API for this including grading by height in the specialization order, and a definition of the pushforward.
- [ ] depends on: #26225
- [ ] depends on: #26259
---
Note there are a couple of things I'm not quite sure about which I've mentioned in the comments, like how I'm not sure how to make the proof of map_locally finite more manageable and so on. Any comment on these (or anything else!) would be greatly appreciated.
[](https://gitpod.io/from-referrer/)
|
t-algebraic-geometry
RFC
merge-conflict
blocked-by-other-PR
|
341/0 |
Mathlib.lean,Mathlib/AlgebraicGeometry/AffineScheme.lean,Mathlib/AlgebraicGeometry/AlgebraicCycle.lean,Mathlib/AlgebraicGeometry/Properties.lean,Mathlib/AlgebraicGeometry/Scheme.lean,Mathlib/Topology/LocallyFinsupp.lean |
6 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
4-61426 4 days ago |
40-1847 1 month ago |
0-366 6 minutes |
27844 |
CBirkbeck author:CBirkbeck |
Breakup eisenstein q exp identity |
---
- [ ] depends on: #27212
- [ ] depends on: #27837
- [ ] depends on: #27839
- [ ] depends on: #27838
- [ ] depends on: #27840
- [ ] depends on: #27841
- [x] depends on: #26016
[](https://gitpod.io/from-referrer/)
|
t-number-theory
merge-conflict
blocked-by-other-PR
|
620/6 |
Mathlib.lean,Mathlib/Analysis/Complex/Exponential.lean,Mathlib/Analysis/Complex/IntegerCompl.lean,Mathlib/Analysis/Complex/SummableUniformlyOn.lean,Mathlib/Analysis/Normed/Module/FiniteDimension.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Cotangent.lean,Mathlib/NumberTheory/ArithmeticFunction.lean,Mathlib/NumberTheory/LSeries/RiemannZeta.lean,Mathlib/NumberTheory/ModularForms/EisensteinSeries/Defs.lean,Mathlib/NumberTheory/ModularForms/EisensteinSeries/QExpansion.lean,Mathlib/NumberTheory/ModularForms/EisensteinSeries/Summable.lean,Mathlib/RingTheory/EuclideanDomain.lean,Mathlib/Topology/Algebra/InfiniteSum/NatInt.lean |
13 |
7 |
['MichaelStollBayreuth', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
4-50778 4 days ago |
15-79636 15 days ago |
0-0 0 seconds |
28796 |
grunweg author:grunweg |
feat: immersions are smooth |
The conventional textbook definition demands that an immersion be smooth.
When asking for the immersion to have local slice charts (as we do), this implies smoothness automatically.
---
- [x] depends on: #28701
- [ ] depends on: #28793
[](https://gitpod.io/from-referrer/)
|
t-differential-geometry
merge-conflict
blocked-by-other-PR
WIP
|
481/7 |
Mathlib.lean,Mathlib/Geometry/Manifold/ChartedSpace.lean,Mathlib/Geometry/Manifold/ContMDiff/Atlas.lean,Mathlib/Geometry/Manifold/IsImmersionEmbedding.lean,Mathlib/Geometry/Manifold/IsManifold/ExtChartAt.lean,Mathlib/Topology/PartialHomeomorph.lean,docs/overview.yaml,docs/references.bib |
8 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
4-48508 4 days ago |
4-48509 4 days ago |
0-1 1 second |
28853 |
grunweg author:grunweg |
feat: product of immersions is an immersion |
---
- [ ] depends on: #28793
- [ ] depends on: ##28796 (for simplicity)
- [x] depends on: #28840
[](https://gitpod.io/from-referrer/)
|
t-differential-geometry
merge-conflict
blocked-by-other-PR
|
640/7 |
Mathlib.lean,Mathlib/Analysis/Calculus/ContDiff/Basic.lean,Mathlib/Geometry/Manifold/ChartedSpace.lean,Mathlib/Geometry/Manifold/ContMDiff/Atlas.lean,Mathlib/Geometry/Manifold/IsImmersionEmbedding.lean,Mathlib/Geometry/Manifold/IsManifold/Basic.lean,Mathlib/Geometry/Manifold/IsManifold/ExtChartAt.lean,Mathlib/Topology/PartialHomeomorph.lean,docs/references.bib |
9 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
4-47988 4 days ago |
4-47989 4 days ago |
0-1911 31 minutes |
28865 |
grunweg author:grunweg |
feat: a map is smooth iff its post-composition with an immersion is |
The continuous case is mostly solved --- except for one detail where I'm not even sure if this is true.
Maybe!, I need to require continuity, at least in general. (Perhaps not for interior points... we'll see!)
A future PR will use this to golf the results in `Icc/Instances.lean`.
---
- [ ] depends on: #28793
- [ ] depends on: #28796
- [ ] depends on: #28853 (for simplicity)
- [ ] depends on: #28905 history bifurcates here: merge that PR first, then rebase this one
[](https://gitpod.io/from-referrer/)
|
t-differential-geometry
merge-conflict
blocked-by-other-PR
WIP
|
1026/7 |
Mathlib.lean,Mathlib/Analysis/Calculus/ContDiff/Basic.lean,Mathlib/Analysis/Calculus/ContDiff/Defs.lean,Mathlib/Geometry/Manifold/ChartedSpace.lean,Mathlib/Geometry/Manifold/ContMDiff/Atlas.lean,Mathlib/Geometry/Manifold/ContMDiff/Defs.lean,Mathlib/Geometry/Manifold/IsImmersionEmbedding.lean,Mathlib/Geometry/Manifold/IsManifold/Basic.lean,Mathlib/Geometry/Manifold/IsManifold/ExtChartAt.lean,Mathlib/Topology/PartialHomeomorph.lean,docs/references.bib,temp_.sh |
12 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
4-47986 4 days ago |
4-47987 4 days ago |
0-11 11 seconds |
28905 |
grunweg author:grunweg |
feat: immersions are locally embeddings |
Hopefully, this can be used for the topological portion of #28865. (That part is not certain yet, the rest works.)
---
TODO: move two helper results about embeddings to their proper place; perhaps even PR separately
- [ ] depends on: #28793
- [ ] depends on: #28796
- [ ] depends on: #28853
[](https://gitpod.io/from-referrer/)
|
merge-conflict
blocked-by-other-PR
|
792/7 |
Mathlib.lean,Mathlib/Analysis/Calculus/ContDiff/Basic.lean,Mathlib/Geometry/Manifold/ChartedSpace.lean,Mathlib/Geometry/Manifold/ContMDiff/Atlas.lean,Mathlib/Geometry/Manifold/IsImmersionEmbedding.lean,Mathlib/Geometry/Manifold/IsManifold/Basic.lean,Mathlib/Geometry/Manifold/IsManifold/ExtChartAt.lean,Mathlib/Topology/PartialHomeomorph.lean,docs/references.bib,temp_.sh |
10 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
4-47985 4 days ago |
4-47986 4 days ago |
0-617 10 minutes |
29077 |
grunweg author:grunweg |
feat(Manifold/Instances/Icc): golf smoothness proof using immersions |
Prove that the inclusion of an interval into the real numbers is a smooth immersion,
and use this to golf the proof that this inclusion is smooth.
TODO: right now, the computation doesn't check out; I need to tweak the charts I have. But that is surely doable.
A future PR will prove it is a smooth embedding.
---
- [ ] depends on: #28865
[](https://gitpod.io/from-referrer/)
|
merge-conflict
blocked-by-other-PR
|
1122/56 |
Mathlib.lean,Mathlib/Analysis/Calculus/ContDiff/Basic.lean,Mathlib/Analysis/Calculus/ContDiff/Defs.lean,Mathlib/Geometry/Manifold/ChartedSpace.lean,Mathlib/Geometry/Manifold/ContMDiff/Atlas.lean,Mathlib/Geometry/Manifold/ContMDiff/Defs.lean,Mathlib/Geometry/Manifold/Instances/Icc.lean,Mathlib/Geometry/Manifold/IsImmersionEmbedding.lean,Mathlib/Geometry/Manifold/IsManifold/Basic.lean,Mathlib/Geometry/Manifold/IsManifold/ExtChartAt.lean,Mathlib/Topology/PartialHomeomorph.lean,docs/references.bib,temp_.sh |
13 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
4-47984 4 days ago |
4-47984 4 days ago |
0-309 5 minutes |
25737 |
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, thanks to the first simplicial identity, composition on the left 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`.
---
- [ ] depends on: #25736
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #21746.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/21746* |
t-algebraic-topology
large-import
t-category-theory
blocked-by-other-PR
|
380/9 |
Mathlib/AlgebraicTopology/SimplexCategory/GeneratorsRelations/NormalForms.lean |
1 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
4-6945 4 days ago |
4-7951 4 days ago |
0-2 2 seconds |
27789 |
staroperator author:staroperator |
feat(ModelTheory): semilinear sets are closed under intersection and set difference |
These are generalizations of the same results on `ℕ ^ k` (in #27414) to any cancellative monoid (e.g. `ℤ ^ k`).
- [ ] depends on: #27414
- [x] depends on: #27786
- [x] depends on: #27787
- [x] depends on: #27955
- [ ] depends on: #29034
- [ ] depends on: #29035
---
[](https://gitpod.io/from-referrer/)
|
t-logic
merge-conflict
blocked-by-other-PR
|
1393/57 |
Mathlib.lean,Mathlib/Algebra/Group/Subgroup/Basic.lean,Mathlib/Algebra/Group/Subgroup/Defs.lean,Mathlib/Algebra/Group/Submonoid/Operations.lean,Mathlib/Data/Set/Prod.lean,Mathlib/GroupTheory/Finiteness.lean,Mathlib/ModelTheory/Arithmetic/Presburger/Semilinear/Basic.lean,Mathlib/ModelTheory/Arithmetic/Presburger/Semilinear/Defs.lean,Mathlib/ModelTheory/Arithmetic/Presburger/Semilinear/Nat.lean,Mathlib/RingTheory/Finiteness/Cardinality.lean,docs/references.bib |
11 |
4 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
3-80220 3 days ago |
16-24997 16 days ago |
0-1510 25 minutes |
27606 |
CBirkbeck author:CBirkbeck |
Eisenstein q exp identity |
---
- [x] depends on: #26016
- [x] depends on: #27212
- [x] depends on: #27837
- [x] depends on: #27839
- [x] depends on: #27840
- [x] depends on: #28690
- [ ] depends on: #27838
- [ ] depends on: #27841
- [ ] depends on: #27844
[](https://gitpod.io/from-referrer/)
|
large-import
merge-conflict
blocked-by-other-PR
|
824/13 |
Mathlib.lean,Mathlib/Analysis/Asymptotics/Lemmas.lean,Mathlib/Analysis/Complex/Exponential.lean,Mathlib/Analysis/Complex/IntegerCompl.lean,Mathlib/Analysis/Complex/Norm.lean,Mathlib/Analysis/Complex/SummableUniformlyOn.lean,Mathlib/Analysis/Normed/Group/Basic.lean,Mathlib/Analysis/Normed/Module/Basic.lean,Mathlib/Analysis/Normed/Module/FiniteDimension.lean,Mathlib/Analysis/RCLike/Basic.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Cotangent.lean,Mathlib/NumberTheory/ArithmeticFunction.lean,Mathlib/NumberTheory/LSeries/RiemannZeta.lean,Mathlib/NumberTheory/ModularForms/EisensteinSeries/Defs.lean,Mathlib/NumberTheory/ModularForms/EisensteinSeries/QExpansion.lean,Mathlib/NumberTheory/ModularForms/EisensteinSeries/Summable.lean,Mathlib/NumberTheory/TsumDivsorsAntidiagonal.lean,Mathlib/Topology/Algebra/InfiniteSum/Basic.lean,Mathlib/Topology/Algebra/InfiniteSum/NatInt.lean |
19 |
6 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
3-80211 3 days ago |
10-46072 10 days ago |
0-0 0 seconds |
26212 |
Thmoas-Guan author:Thmoas-Guan |
feat(Algebra): the Rees theorem for depth |
In this PR we proved the Rees theorem for depth.
Co-authored-by: Hu Yongle
---
- [ ] depends on: #26211
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebra
blocked-by-other-PR
label:t-algebra$ |
306/5 |
Mathlib/Algebra/Category/Grp/Preadditive.lean,Mathlib/RingTheory/Ideal/AssociatedPrime/Localization.lean,Mathlib/RingTheory/Regular/Category.lean,Mathlib/RingTheory/Regular/Depth.lean |
4 |
n/a |
['Thmoas-Guan', 'github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
3-67944 3 days ago |
unknown |
unknown |
26213 |
Thmoas-Guan author:Thmoas-Guan |
feat(Algebra): Ext iso quotient regular sequence |
In this PR defined the `addequiv` between `Ext M N k` and `N =>[R] M/ rs * M` where `rs` is a regular sequence of length `k`
Co-authored-by: Hu Yongle
Co-authored-by: Wang Jingting
---
- [ ] depends on: #26212
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebra
blocked-by-other-PR
label:t-algebra$ |
366/5 |
Mathlib/Algebra/Category/Grp/Preadditive.lean,Mathlib/RingTheory/Ideal/AssociatedPrime/Localization.lean,Mathlib/RingTheory/Regular/Category.lean,Mathlib/RingTheory/Regular/Depth.lean |
4 |
n/a |
['Thmoas-Guan', 'github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
3-67851 3 days ago |
unknown |
unknown |
26214 |
Thmoas-Guan author:Thmoas-Guan |
feat(Algebra): definition of depth |
In this PR, we defined the depth of two modules as the minimal order of nonvanishing `Ext` and the `I-depth` for ideal `I` and some basic properties. Including the equivalence of the two in the condition of rees theorem.
---
- [ ] depends on: #26212
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebra
blocked-by-other-PR
label:t-algebra$ |
694/5 |
Mathlib/Algebra/Category/Grp/Preadditive.lean,Mathlib/RingTheory/Ideal/AssociatedPrime/Localization.lean,Mathlib/RingTheory/Regular/Category.lean,Mathlib/RingTheory/Regular/Depth.lean |
4 |
n/a |
['Thmoas-Guan', 'github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
3-67787 3 days ago |
unknown |
unknown |
26217 |
Thmoas-Guan author:Thmoas-Guan |
feat(Algebra): Ischebeck theorem |
This PR mainly proved the Ischbecke theorem, stating that `depth(N,M)` is greater or equal to `depth(M) - dim(N)` for finitely generated module `N, M` over local ring.
---
- [ ] depends on: #26214
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebra
blocked-by-other-PR
label:t-algebra$ |
1051/5 |
Mathlib.lean,Mathlib/Algebra/Category/Grp/Preadditive.lean,Mathlib/RingTheory/Ideal/AssociatedPrime/Localization.lean,Mathlib/RingTheory/Regular/Category.lean,Mathlib/RingTheory/Regular/Depth.lean,Mathlib/RingTheory/Regular/Ischebeck.lean |
6 |
n/a |
['Thmoas-Guan', 'github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
3-67527 3 days ago |
unknown |
unknown |
26215 |
Thmoas-Guan author:Thmoas-Guan |
feat(Algebra): Auslander-Buchsbaum theorem |
This PR mainly proved the Auslander-Buchsbaum theorem stating for a noetherian local ring `R` and a finitely generated `R` module `M` , `proj.dim(M) + depth(M) = depth(R)`.
Co-authored-by: Yongle Hu
---
- [ ] depends on: #26214
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebra
blocked-by-other-PR
label:t-algebra$ |
1198/5 |
Mathlib.lean,Mathlib/Algebra/Category/Grp/Preadditive.lean,Mathlib/RingTheory/Ideal/AssociatedPrime/Localization.lean,Mathlib/RingTheory/Regular/AuslanderBuchsbaum.lean,Mathlib/RingTheory/Regular/Category.lean,Mathlib/RingTheory/Regular/Depth.lean |
6 |
n/a |
['Thmoas-Guan', 'github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
3-67289 3 days ago |
unknown |
unknown |
29447 |
j-loreaux author:j-loreaux |
chore(Analysis/NormedSpace/HahnBanach): move and split files |
This moves or splits the files in `Analysis/NormedSpace/HahnBanach/` accordingly:
- `Separation` → `Analysis/LocallyConvex/Separation`
- `Extension` → `Analysis/Normed/Module/HahnBanach/Extension`
- `SeparatingDual`: split, mostly in `Analysis/LocallyConvex/SeparatingDual`, but a few completeness results are sent to `Analysis/Normed/Module/HahnBanach/Completeness`.
The split allows us to significantly reduce the imports of `SeparatingDual`, albeit with a new proof that a normed space over `RCLike 𝕜` has a separating dual. Here we use the geometric Hahn-Banach theorem instead of the analytic one.
This is part of #28698 to migrate the material in `Analysis/NormedSpace/` to other locations.
---
- [ ] depends on: #29445
[](https://gitpod.io/from-referrer/)
|
file-removed
merge-conflict
blocked-by-other-PR
|
291/235 |
Counterexamples/Phillips.lean,Mathlib.lean,Mathlib/Analysis/Calculus/ParametricIntegral.lean,Mathlib/Analysis/Convex/Cone/Dual.lean,Mathlib/Analysis/Convex/KreinMilman.lean,Mathlib/Analysis/LocallyConvex/SeparatingDual.lean,Mathlib/Analysis/LocallyConvex/Separation.lean,Mathlib/Analysis/LocallyConvex/WeakOperatorTopology.lean,Mathlib/Analysis/LocallyConvex/WeakSpace.lean,Mathlib/Analysis/Normed/Module/Dual.lean,Mathlib/Analysis/Normed/Module/HahnBanach/Completeness.lean,Mathlib/Analysis/Normed/Module/HahnBanach/Extension.lean,Mathlib/Analysis/Normed/Module/RCLike/Extend.lean,Mathlib/Analysis/NormedSpace/Extend.lean,Mathlib/Analysis/RCLike/Extend.lean,Mathlib/MeasureTheory/Integral/Bochner/ContinuousLinearMap.lean |
16 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
3-15862 3 days ago |
3-15863 3 days ago |
0-259 4 minutes |
29472 |
chrisflav author:chrisflav |
feat(CategoryTheory/Sites): functoriality of precoverages and `0`-hypercovers |
---
- [ ] depends on: #28614
[](https://gitpod.io/from-referrer/)
|
t-category-theory
merge-conflict
blocked-by-other-PR
|
109/0 |
Mathlib/CategoryTheory/Sites/Precoverage.lean,Mathlib/CategoryTheory/Sites/Sieves.lean,Mathlib/CategoryTheory/Sites/ZeroHypercover.lean |
3 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
3-15857 3 days ago |
3-15858 3 days ago |
0-1236 20 minutes |
28683 |
Thmoas-Guan author:Thmoas-Guan |
feat(RingTheory) : regular local ring is domain |
In this PR, we proved for a regular local ring `R`,
1 : for a finite set `S` in the maximal Ideal of `R`, it can be extended to a regular system of parameters iff they are linear independent in the cotangent space iff `R/span S` is regular local ring of dimesion `dim R - |S|`
2 : is domain
3 : regular system of parameter form regular sequence.
---
- [ ] depends on: #28682
- [ ] depends on: #28582
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
blocked-by-other-PR
WIP
|
461/0 |
Mathlib.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/RingTheory/RegularLocalRing/Basic.lean,Mathlib/RingTheory/RegularLocalRing/Defs.lean |
4 |
3 |
['Thmoas-Guan', 'github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
3-11015 3 days ago |
24-6808 24 days ago |
0-111 1 minute |
28684 |
Thmoas-Guan author:Thmoas-Guan |
feat(RingTheory) : definition of regular ring |
In this PR, we define regular ring as every localization is regular local ring, and proved polynomial over regular ring is regular.
---
- [ ] depends on: #28682
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
blocked-by-other-PR
WIP
|
306/0 |
Mathlib.lean,Mathlib/RingTheory/RegularLocalRing/Defs.lean,Mathlib/RingTheory/RegularLocalRing/RegularRing.lean |
3 |
3 |
['Thmoas-Guan', 'github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
3-10922 3 days ago |
24-6809 24 days ago |
0-153 2 minutes |
28804 |
grunweg author:grunweg |
feat: a few more tactic linters |
All analysis passes in this list have been suggested [on zulip](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Tactic.20analysis.20framework/with/535766713).
---
Untested, so may not work yet.
- [ ] depends on: #28802
[](https://gitpod.io/from-referrer/)
|
t-meta
merge-conflict
blocked-by-other-PR
|
204/26 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/TacticAnalysis/Declarations.lean,Mathlib/Tactic/TacticAnalysis/FunProp.lean,Mathlib/Tactic/TacticAnalysis/Misc.lean,MathlibTest/TacticAnalysis2.lean |
6 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
3-7129 3 days ago |
3-7130 3 days ago |
0-705 11 minutes |
26216 |
Thmoas-Guan author:Thmoas-Guan |
feat(Algebra): depth of QuotSMulTop |
In this PR, we proved for a local ring `R` and a finitely generated `R` module `M N`, `IsSMulRegular M x` and `x ∈ Module.annihilator R N`, then `depth(N, M/xM) + 1 = depth(N, M)`, and its corollary for quotient regular seqence.
---
- [ ] depends on: #26214
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebra
blocked-by-other-PR
label:t-algebra$ |
987/5 |
Mathlib/Algebra/Category/Grp/Preadditive.lean,Mathlib/RingTheory/Ideal/AssociatedPrime/Localization.lean,Mathlib/RingTheory/Regular/Category.lean,Mathlib/RingTheory/Regular/Depth.lean |
4 |
n/a |
['Thmoas-Guan', 'github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
3-5538 3 days ago |
unknown |
unknown |
26218 |
Thmoas-Guan author:Thmoas-Guan |
feat(Algebra): definition of cohen macaulay |
In this PR, we added the definition of CM module, CM local ring (extending local ring), and CM ring.
We also proved Theorem 30, Chater 6, _Commutative Algebra_, Matsumura.
---
- [ ] depends on: #26219
- [ ] depends on: #26217
- [ ] depends on: #26216
- [ ] depends on: #28582
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebra
blocked-by-other-PR
label:t-algebra$ |
2212/40 |
Mathlib.lean,Mathlib/Algebra/Category/Grp/Preadditive.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/LinearAlgebra/Quotient/Basic.lean,Mathlib/RingTheory/CohenMacaulay/Basic.lean,Mathlib/RingTheory/Ideal/AssociatedPrime/Localization.lean,Mathlib/RingTheory/Ideal/MinimalPrime/Localization.lean,Mathlib/RingTheory/Jacobson/Ideal.lean,Mathlib/RingTheory/KrullDimension/Module.lean,Mathlib/RingTheory/KrullDimension/Regular.lean,Mathlib/RingTheory/LocalRing/MaximalIdeal/Basic.lean,Mathlib/RingTheory/Nakayama.lean,Mathlib/RingTheory/Regular/Category.lean,Mathlib/RingTheory/Regular/Depth.lean,Mathlib/RingTheory/Regular/Ischebeck.lean,Mathlib/RingTheory/Support.lean |
16 |
n/a |
['Thmoas-Guan', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
3-5439 3 days ago |
unknown |
unknown |
26245 |
Thmoas-Guan author:Thmoas-Guan |
feat(Algebra): cohen macaulay local ring is catenary |
We prove Cohen Macaulay local ring is catenary.
Following Theorem 31, Chater 6, _Commutative Algebra_, Matsumura
---
- [ ] depends on: #26218
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebra
blocked-by-other-PR
WIP
label:t-algebra$ |
2599/40 |
Mathlib.lean,Mathlib/Algebra/Category/Grp/Preadditive.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/LinearAlgebra/Quotient/Basic.lean,Mathlib/RingTheory/CohenMacaulay/Basic.lean,Mathlib/RingTheory/CohenMacaulay/Catenary.lean,Mathlib/RingTheory/Ideal/AssociatedPrime/Localization.lean,Mathlib/RingTheory/Ideal/MinimalPrime/Localization.lean,Mathlib/RingTheory/Jacobson/Ideal.lean,Mathlib/RingTheory/KrullDimension/Module.lean,Mathlib/RingTheory/KrullDimension/Regular.lean,Mathlib/RingTheory/LocalRing/MaximalIdeal/Basic.lean,Mathlib/RingTheory/Nakayama.lean,Mathlib/RingTheory/Regular/Category.lean,Mathlib/RingTheory/Regular/Depth.lean,Mathlib/RingTheory/Regular/Ischebeck.lean,Mathlib/RingTheory/Support.lean |
17 |
n/a |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
3-5020 3 days ago |
unknown |
unknown |
26957 |
Thmoas-Guan author:Thmoas-Guan |
feat(Algebra): unmixed thm of Cohen-Macaulay ring |
In this PR we proved for a (comm)ring `R`, `R` is Cohen-Macaulay ring iff the unmixed theorem holds (for every ideal `I` of height `r` generated by `r` elements, all associated primes of `R/I` have height `r` )
---
- [ ] depends on: #26245
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebra
blocked-by-other-PR
label:t-algebra$ |
2773/40 |
Mathlib.lean,Mathlib/Algebra/Category/Grp/Preadditive.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/LinearAlgebra/Quotient/Basic.lean,Mathlib/RingTheory/CohenMacaulay/Basic.lean,Mathlib/RingTheory/CohenMacaulay/Catenary.lean,Mathlib/RingTheory/CohenMacaulay/Unmixed.lean,Mathlib/RingTheory/Ideal/AssociatedPrime/Localization.lean,Mathlib/RingTheory/Ideal/MinimalPrime/Localization.lean,Mathlib/RingTheory/Jacobson/Ideal.lean,Mathlib/RingTheory/KrullDimension/Module.lean,Mathlib/RingTheory/KrullDimension/Regular.lean,Mathlib/RingTheory/LocalRing/MaximalIdeal/Basic.lean,Mathlib/RingTheory/Nakayama.lean,Mathlib/RingTheory/Regular/Category.lean,Mathlib/RingTheory/Regular/Depth.lean,Mathlib/RingTheory/Regular/Ischebeck.lean,Mathlib/RingTheory/Support.lean |
18 |
n/a |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
3-5012 3 days ago |
unknown |
unknown |
29508 |
zhuyizheng author:zhuyizheng |
feat(MeasureTheory): FTC and integration by parts for absolutely continuous functions |
Prove Fundamental Theorem of Calculus and integration by parts for absolutely continuous functions. Part of originally planned #29092.
---
- [ ] depends on: #29503
- [ ] depends on: #29507
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-measure-probability
blocked-by-other-PR
|
1378/0 |
Mathlib.lean,Mathlib/Analysis/Calculus/Deriv/Slope.lean,Mathlib/MeasureTheory/Function/AbsolutelyContinuous.lean,Mathlib/MeasureTheory/Integral/IntervalIntegral/AbsContFunc.lean,Mathlib/MeasureTheory/Integral/IntervalIntegral/DerivIntegrable.lean,Mathlib/MeasureTheory/Integral/IntervalIntegral/LebesgueDifferetiationThm.lean,Mathlib/Topology/EMetricSpace/BoundedVariation.lean |
7 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
2-65926 2 days ago |
2-65926 2 days ago |
0-261 4 minutes |
29507 |
zhuyizheng author:zhuyizheng |
feat(MeasureTheory): derivative integrable functions |
Part of originally planned #29092. We prove that:
* If `f` is monotone on `a..b`, then `f'` is interval integrable on `a..b`.
* If `f` has bounded variation on `a..b`, then `f'` is interval integrable on `a..b`.
* If `f` is absolutely continuous on `a..b`, then `f'` exists a.e. on `a..b` and is interval
integrable on `a..b`.
---
- [ ] depends on: #29504
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-measure-probability
blocked-by-other-PR
|
647/0 |
Mathlib.lean,Mathlib/MeasureTheory/Function/AbsolutelyContinuous.lean,Mathlib/MeasureTheory/Integral/IntervalIntegral/DerivIntegrable.lean,Mathlib/Topology/EMetricSpace/BoundedVariation.lean |
4 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
2-65888 2 days ago |
2-65888 2 days ago |
0-324 5 minutes |
28968 |
linesthatinterlace author:linesthatinterlace |
refactor(Order/Hom/Basic): Replace `abbrev` with `def` in OrderEmbedding and OrderIso |
---
- [ ] depends on: #28944
[](https://gitpod.io/from-referrer/)
|
merge-conflict
blocked-by-other-PR
|
258/200 |
Mathlib/Data/Sum/Order.lean,Mathlib/Order/FixedPoints.lean,Mathlib/Order/Hom/Basic.lean,Mathlib/Order/Hom/Order.lean |
4 |
5 |
['YaelDillies', 'github-actions', 'linesthatinterlace', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
b-mehta and linesthatinterlace assignee:b-mehta assignee:linesthatinterlace |
2-64502 2 days ago |
2-64503 2 days ago |
0-0 0 seconds |
29116 |
scholzhannah author:scholzhannah |
chore(Topology/PartialHomeomorph): add module deprecation |
This is the follow-up PR of #29113 adding the deprecated module after the file was renamed.
---
- [ ] depends on: #29113
[](https://gitpod.io/from-referrer/)
|
blocked-by-other-PR |
2500/2260 |
Mathlib.lean,Mathlib/Analysis/Analytic/Inverse.lean,Mathlib/Analysis/Asymptotics/Defs.lean,Mathlib/Analysis/Asymptotics/Lemmas.lean,Mathlib/Analysis/Calculus/ContDiff/Operations.lean,Mathlib/Analysis/Calculus/Deriv/Inverse.lean,Mathlib/Analysis/Calculus/FDeriv/Analytic.lean,Mathlib/Analysis/Calculus/FDeriv/Equiv.lean,Mathlib/Analysis/Calculus/Implicit.lean,Mathlib/Analysis/Calculus/InverseFunctionTheorem/ApproximatesLinearOn.lean,Mathlib/Analysis/Calculus/InverseFunctionTheorem/ContDiff.lean,Mathlib/Analysis/Calculus/InverseFunctionTheorem/FDeriv.lean,Mathlib/Analysis/Complex/Tietze.lean,Mathlib/Analysis/Complex/UpperHalfPlane/Topology.lean,Mathlib/Analysis/InnerProductSpace/Calculus.lean,Mathlib/Analysis/Normed/Module/Ball/Homeomorph.lean,Mathlib/Analysis/SpecialFunctions/Arsinh.lean,Mathlib/Analysis/SpecialFunctions/Complex/LogDeriv.lean,Mathlib/Analysis/SpecialFunctions/Log/Basic.lean,Mathlib/Analysis/SpecialFunctions/PolarCoord.lean,Mathlib/Analysis/SpecialFunctions/Sqrt.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Arctan.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Inverse.lean,Mathlib/Deprecated/AnalyticManifold.lean,Mathlib/Geometry/Manifold/ChartedSpace.lean,Mathlib/Geometry/Manifold/ConformalGroupoid.lean,Mathlib/Geometry/Manifold/ContMDiff/Atlas.lean,Mathlib/Geometry/Manifold/ContMDiff/Basic.lean,Mathlib/Geometry/Manifold/ContMDiff/Defs.lean,Mathlib/Geometry/Manifold/ContMDiffMFDeriv.lean,Mathlib/Geometry/Manifold/Diffeomorph.lean,Mathlib/Geometry/Manifold/Instances/Icc.lean,Mathlib/Geometry/Manifold/Instances/Real.lean,Mathlib/Geometry/Manifold/Instances/Sphere.lean,Mathlib/Geometry/Manifold/IsManifold/Basic.lean,Mathlib/Geometry/Manifold/IsManifold/ExtChartAt.lean,Mathlib/Geometry/Manifold/IsManifold/InteriorBoundary.lean,Mathlib/Geometry/Manifold/LocalDiffeomorph.lean,Mathlib/Geometry/Manifold/LocalInvariantProperties.lean,Mathlib/Geometry/Manifold/MFDeriv/Atlas.lean,Mathlib/Geometry/Manifold/MFDeriv/Basic.lean,Mathlib/Geometry/Manifold/MFDeriv/Defs.lean,Mathlib/Geometry/Manifold/MFDeriv/Tangent.lean,Mathlib/Geometry/Manifold/MFDeriv/UniqueDifferential.lean,Mathlib/Geometry/Manifold/PartitionOfUnity.lean,Mathlib/Geometry/Manifold/VectorBundle/Basic.lean,Mathlib/Geometry/Manifold/VectorBundle/FiberwiseLinear.lean,Mathlib/Geometry/Manifold/VectorBundle/Hom.lean,Mathlib/Geometry/Manifold/VectorBundle/MDifferentiable.lean,Mathlib/Geometry/Manifold/VectorBundle/Tangent.lean,Mathlib/Logic/Equiv/PartialEquiv.lean,Mathlib/MeasureTheory/Function/Jacobian.lean,Mathlib/NumberTheory/ModularForms/EisensteinSeries/UniformConvergence.lean,Mathlib/NumberTheory/NumberField/CanonicalEmbedding/NormLeOne.lean,Mathlib/NumberTheory/NumberField/CanonicalEmbedding/PolarCoord.lean,Mathlib/Topology/Covering.lean,Mathlib/Topology/FiberBundle/Basic.lean,Mathlib/Topology/FiberBundle/Constructions.lean,Mathlib/Topology/FiberBundle/Trivialization.lean,Mathlib/Topology/Instances/AddCircle/Defs.lean,Mathlib/Topology/IsLocalHomeomorph.lean,Mathlib/Topology/OpenPartialHomeomorph.lean,Mathlib/Topology/PartialHomeomorph.lean,Mathlib/Topology/VectorBundle/Basic.lean,MathlibTest/MfldSetTac.lean |
65 |
7 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
2-59540 2 days ago |
2-59558 2 days ago |
0-509 8 minutes |
28291 |
vasnesterov author:vasnesterov |
feat(Tactic): tactic for computing asymptotics of real functions |
It's an auxiliary PR which implements the entire `compute_asymptotics` tactic. I will split it into multiple small PRs if it is decided that we will merge it.
---
In this PR I implement the `compute_asymptotics` tactic. Its purpose is to compute asymptotics of functions from `ℝ` to `ℝ`. So far it is able to compute the limit of any function constructed using arithmetic operations (`+`, `-`, `*`, `/`, inversion), powers with constant real exponent, logarithms, and exponents.
```lean
import Mathlib.Tactic.ComputeAsymptotics
open Real Filter Topology Asymptotics
example : Tendsto (fun (x : ℝ) ↦ (1 + 6 * x⁻¹) ^ (7 * x)) atTop (𝓝 (exp 42)) := by
compute_asymptotics
example : (fun x ↦ x - 1 - log x) ~[𝓝[≠] 1] (fun x ↦ (x - 1) ^ 2 / 2) := by
compute_asymptotics
example (a b : ℝ) (h : a < b) :
(fun x ↦ (x + x * log x) ^ a) =O[atTop] (fun x ↦ (x / log x) ^ b) := by
compute_asymptotics
example :
(fun x ↦ log x) =o[𝓝[>] 0] (fun x ↦ Real.pi / (exp (Real.log 2 * x) - 1)) := by
compute_asymptotics
```
For more examples see `compute_asymptotics.lean` in tests.
### TODO
* `compute_limit%` elaborator that computes the limit and returns a proof.
* Support different domains (`ℕ`, `ℤ`, `ℚ`).
* Support trigonometric functions and Gamma-function.
### References
I am basically implementing [this article](https://www21.in.tum.de/~eberlm/pdfs/real_asymp.pdf) about computing asymptotics in Isabelle by Manuel Eberl.
- [ ] depends on: #23831
- [ ] depends on: #26120
- [ ] depends on: #28874
[](https://gitpod.io/from-referrer/)
|
t-analysis
t-meta
merge-conflict
blocked-by-other-PR
WIP
|
17130/340 |
Mathlib.lean,Mathlib/Analysis/Analytic/Basic.lean,Mathlib/Analysis/Analytic/OfScalars.lean,Mathlib/Analysis/Calculus/FDeriv/Analytic.lean,Mathlib/Analysis/Calculus/FormalMultilinearSeries.lean,Mathlib/Analysis/Calculus/IteratedDeriv/Defs.lean,Mathlib/Analysis/SpecialFunctions/Complex/Analytic.lean,Mathlib/Data/Nat/Factorial/Basic.lean,Mathlib/Data/Seq/Parallel.lean,Mathlib/Data/Seq/Seq.lean,Mathlib/Data/Set/Pointwise/Interval.lean,Mathlib/Tactic.lean,Mathlib/Tactic/ComputeAsymptotics.lean,Mathlib/Tactic/ComputeAsymptotics/Lemmas.lean,Mathlib/Tactic/ComputeAsymptotics/Meta/BasisM.lean,Mathlib/Tactic/ComputeAsymptotics/Meta/CompareMS.lean,Mathlib/Tactic/ComputeAsymptotics/Meta/CompareReal.lean,Mathlib/Tactic/ComputeAsymptotics/Meta/ConstSimp.lean,Mathlib/Tactic/ComputeAsymptotics/Meta/ConstSimpAttribute.lean,Mathlib/Tactic/ComputeAsymptotics/Meta/Defs.lean,Mathlib/Tactic/ComputeAsymptotics/Meta/Exp.lean,Mathlib/Tactic/ComputeAsymptotics/Meta/LeadingTerm.lean,Mathlib/Tactic/ComputeAsymptotics/Meta/Log.lean,Mathlib/Tactic/ComputeAsymptotics/Meta/MS.lean,Mathlib/Tactic/ComputeAsymptotics/Meta/Misc.lean,Mathlib/Tactic/ComputeAsymptotics/Meta/Normalization.lean,Mathlib/Tactic/ComputeAsymptotics/Meta/Trimming.lean,Mathlib/Tactic/ComputeAsymptotics/Multiseries.lean,Mathlib/Tactic/ComputeAsymptotics/Multiseries/Basic.lean,Mathlib/Tactic/ComputeAsymptotics/Multiseries/Basis.lean,Mathlib/Tactic/ComputeAsymptotics/Multiseries/Defs.lean,Mathlib/Tactic/ComputeAsymptotics/Multiseries/LeadingTerm.lean,Mathlib/Tactic/ComputeAsymptotics/Multiseries/LogBasis.lean,Mathlib/Tactic/ComputeAsymptotics/Multiseries/Operations.lean,Mathlib/Tactic/ComputeAsymptotics/Multiseries/Operations/Add.lean,Mathlib/Tactic/ComputeAsymptotics/Multiseries/Operations/Basic.lean,Mathlib/Tactic/ComputeAsymptotics/Multiseries/Operations/Exp.lean,Mathlib/Tactic/ComputeAsymptotics/Multiseries/Operations/ForPow.lean,Mathlib/Tactic/ComputeAsymptotics/Multiseries/Operations/Inv.lean,Mathlib/Tactic/ComputeAsymptotics/Multiseries/Operations/Log.lean,Mathlib/Tactic/ComputeAsymptotics/Multiseries/Operations/Merge.lean,Mathlib/Tactic/ComputeAsymptotics/Multiseries/Operations/Mul.lean,Mathlib/Tactic/ComputeAsymptotics/Multiseries/Operations/Pow.lean,Mathlib/Tactic/ComputeAsymptotics/Multiseries/Operations/Powser.lean,Mathlib/Tactic/ComputeAsymptotics/Multiseries/Term.lean,Mathlib/Tactic/ComputeAsymptotics/Multiseries/Trimming.lean,Mathlib/Tactic/NormNum/NatFactorial.lean,Mathlib/Topology/Algebra/Order/Field.lean,MathlibTest/compute_asymptotics.lean,MathlibTest/kek.lean,scripts/README.md,scripts/migrate_to_fork.py,scripts/noshake.json |
53 |
1 |
['mathlib4-dependent-issues-bot'] |
nobody |
2-47950 2 days ago |
31-76647 1 month ago |
0-54 54 seconds |
29533 |
Thmoas-Guan author:Thmoas-Guan |
feat(Algebra): maximal Cohen Macaulay module |
In this PR, we defined the concept of maximal Cohen Macaulay module, and proved that finitely generated maximal Cohen Macaulay module over regular local ring is free.
---
- [ ] depends on: #28683
- [ ] depends on: #26218
[](https://gitpod.io/from-referrer/)
|
large-import
blocked-by-other-PR
|
2840/40 |
Mathlib.lean,Mathlib/Algebra/Category/Grp/Preadditive.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/LinearAlgebra/Quotient/Basic.lean,Mathlib/RingTheory/CohenMacaulay/Basic.lean,Mathlib/RingTheory/CohenMacaulay/Maximal.lean,Mathlib/RingTheory/Ideal/AssociatedPrime/Localization.lean,Mathlib/RingTheory/Ideal/MinimalPrime/Localization.lean,Mathlib/RingTheory/Jacobson/Ideal.lean,Mathlib/RingTheory/KrullDimension/Module.lean,Mathlib/RingTheory/KrullDimension/Regular.lean,Mathlib/RingTheory/LocalRing/MaximalIdeal/Basic.lean,Mathlib/RingTheory/Nakayama.lean,Mathlib/RingTheory/Regular/Category.lean,Mathlib/RingTheory/Regular/Depth.lean,Mathlib/RingTheory/Regular/Ischebeck.lean,Mathlib/RingTheory/RegularLocalRing/Basic.lean,Mathlib/RingTheory/RegularLocalRing/Defs.lean,Mathlib/RingTheory/Support.lean |
19 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
2-31900 2 days ago |
2-31989 2 days ago* |
2-31970 2 days* |
29000 |
JovanGerb author:JovanGerb |
feat(Tactic/Push): add basic tags and tests |
This PR adds basic `@[push]` tags, and expands the `push` test file.
---
- [ ] depends on: #21965
[](https://gitpod.io/from-referrer/)
|
merge-conflict
blocked-by-other-PR
|
623/210 |
Mathlib.lean,Mathlib/Algebra/Lie/Weights/Killing.lean,Mathlib/Algebra/Notation/Pi/Defs.lean,Mathlib/Analysis/SpecialFunctions/Log/Basic.lean,Mathlib/Combinatorics/SimpleGraph/Coloring.lean,Mathlib/Combinatorics/SimpleGraph/Extremal/Basic.lean,Mathlib/Data/Nat/Basic.lean,Mathlib/Data/Nat/Cast/Basic.lean,Mathlib/Data/Set/Basic.lean,Mathlib/Data/Set/Insert.lean,Mathlib/Data/Set/Operations.lean,Mathlib/Order/Defs/LinearOrder.lean,Mathlib/RingTheory/AlgebraicIndependent/TranscendenceBasis.lean,Mathlib/RingTheory/HahnSeries/Lex.lean,Mathlib/RingTheory/Multiplicity.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Push.lean,Mathlib/Tactic/Push/Attr.lean,Mathlib/Topology/Algebra/IsUniformGroup/Basic.lean,MathlibTest/push.lean,MathlibTest/push_neg.lean,scripts/noshake.json |
22 |
4 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
2-19762 2 days ago |
2-19762 2 days ago |
0-131 2 minutes |
29519 |
joelriou author:joelriou |
feat(CategoryTheory): strong generators |
In this PR, we introduce a condition `IsStrongGenerator S` on a set `S` of objects in a category `C` which is stronger than `IsSeparating S` as we also require that for any proper subobject `A ⊂ X`, there exists a morphism `G ⟶ X` from an
object in `S` which does not factor through `A`.
In case coproducts exists, we give a characterization of `IsStrongSeparator S` (resp. `IsSeparating S`) in terms of the existence, for each object `X : C` of an extremal epi (resp. epi) to `X` from a coproduct of objects in `S`.
In future works, this shall be used in order to characterize locally `κ`-presentable categories as cocomplete categories that have a strong generator consisting of `κ`-presentable objects.
---
- [ ] depends on: #29518
[](https://gitpod.io/from-referrer/)
|
t-category-theory
blocked-by-other-PR
WIP
|
281/0 |
Mathlib.lean,Mathlib/CategoryTheory/ExtremalEpi.lean,Mathlib/CategoryTheory/Generator/StrongGenerator.lean |
3 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
2-9153 2 days ago |
2-37905 2 days ago |
0-2 2 seconds |
29543 |
joelriou author:joelriou |
feat(CategoryTheory): a set S of objects is a strong generator if any object is a colimit of objects in S |
---
- [ ] depends on: #29519
- [ ] depends on: #29518
[](https://gitpod.io/from-referrer/)
|
large-import
t-category-theory
blocked-by-other-PR
|
337/2 |
Mathlib.lean,Mathlib/CategoryTheory/ExtremalEpi.lean,Mathlib/CategoryTheory/Generator/StrongGenerator.lean,Mathlib/CategoryTheory/Presentable/CardinalFilteredPresentation.lean |
4 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
2-7568 2 days ago |
2-7569 2 days ago |
0-1700 28 minutes |
23177 |
faenuccio author:faenuccio |
feat: more lemmas about ordered groups with zero |
We add some order properties (mainly some `lt`) for types of the form `WithZero α`.
Co-authored-by: María Inés de Frutos Fernández
---
- [x] depends on: #26665
- [x] depends on: #26724
- [x] depends on: #26761
- [x] depends on: #26762
- [x] depends on: #26763
- [ ] depends on: #26777 |
large-import
t-order
awaiting-CI
blocked-by-other-PR
WIP
|
13/1 |
Mathlib/Algebra/Order/GroupWithZero/Unbundled/Basic.lean |
1 |
46 |
['Vierkantor', 'YaelDillies', 'faenuccio', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
1-82360 1 day ago |
38-66993 1 month ago |
5-22106 5 days |
29555 |
RemyDegenne author:RemyDegenne |
feat(Probability): `condDistrib` lemmas |
From the LeanBandits project.
---
- [ ] depends on: #29552
[](https://gitpod.io/from-referrer/)
|
t-measure-probability
blocked-by-other-PR
|
150/2 |
Mathlib/Probability/ConditionalProbability.lean,Mathlib/Probability/Kernel/Composition/Lemmas.lean,Mathlib/Probability/Kernel/Composition/MeasureComp.lean,Mathlib/Probability/Kernel/Composition/ParallelComp.lean,Mathlib/Probability/Kernel/Composition/Prod.lean,Mathlib/Probability/Kernel/CondDistrib.lean,Mathlib/Probability/Kernel/Condexp.lean |
7 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
1-81502 1 day ago |
1-81503 1 day ago |
0-1004 16 minutes |
29557 |
Thmoas-Guan author:Thmoas-Guan |
feat(Algebra): finite projective dimension of regular |
In this PR, we proved every finitely generated module over regular local ring has finite projective dimension. With this and Auslander Buchsbaum theorem, we can obtain the global dimension of regular local ring is equal to its krull dimension.
---
- [ ] depends on: #29533
- [ ] depends on: #26215
[](https://gitpod.io/from-referrer/)
|
large-import
blocked-by-other-PR
|
3430/40 |
Mathlib.lean,Mathlib/Algebra/Category/Grp/Preadditive.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/LinearAlgebra/Quotient/Basic.lean,Mathlib/RingTheory/CohenMacaulay/Basic.lean,Mathlib/RingTheory/CohenMacaulay/Maximal.lean,Mathlib/RingTheory/Ideal/AssociatedPrime/Localization.lean,Mathlib/RingTheory/Ideal/MinimalPrime/Localization.lean,Mathlib/RingTheory/Jacobson/Ideal.lean,Mathlib/RingTheory/KrullDimension/Module.lean,Mathlib/RingTheory/KrullDimension/Regular.lean,Mathlib/RingTheory/LocalRing/MaximalIdeal/Basic.lean,Mathlib/RingTheory/Nakayama.lean,Mathlib/RingTheory/Regular/AuslanderBuchsbaum.lean,Mathlib/RingTheory/Regular/Category.lean,Mathlib/RingTheory/Regular/Depth.lean,Mathlib/RingTheory/Regular/Ischebeck.lean,Mathlib/RingTheory/RegularLocalRing/Basic.lean,Mathlib/RingTheory/RegularLocalRing/Defs.lean,Mathlib/RingTheory/RegularLocalRing/GlobalDimension.lean,Mathlib/RingTheory/Support.lean |
21 |
n/a |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
1-73280 1 day ago |
unknown |
unknown |
26651 |
loefflerd author:loefflerd |
WIP: modular forms for subgroups not contained in SL2Z |
This PR generalizes (some of) the modular forms files to allow the level to be any subgroup of GL(2, R), not necessarily
the image of a subgroup of SL(2, Z). Intended applications include defining Hecke operators.
---
- [x] depends on: #26811
- [x] depends on: #28552
- [ ] depends on: #29327
- [ ] depends on: #29560
[](https://gitpod.io/from-referrer/)
|
t-number-theory
blocked-by-other-PR
WIP
|
889/310 |
Mathlib.lean,Mathlib/Analysis/Complex/UpperHalfPlane/FunctionsBoundedAtInfty.lean,Mathlib/Analysis/Complex/UpperHalfPlane/MoebiusAction.lean,Mathlib/LinearAlgebra/Matrix/GeneralLinearGroup/Defs.lean,Mathlib/NumberTheory/ModularForms/ArithmeticSubgroups.lean,Mathlib/NumberTheory/ModularForms/Basic.lean,Mathlib/NumberTheory/ModularForms/BoundedAtCusp.lean,Mathlib/NumberTheory/ModularForms/CongruenceSubgroups.lean,Mathlib/NumberTheory/ModularForms/Cusps.lean,Mathlib/NumberTheory/ModularForms/EisensteinSeries/Basic.lean,Mathlib/NumberTheory/ModularForms/EisensteinSeries/Defs.lean,Mathlib/NumberTheory/ModularForms/Identities.lean,Mathlib/NumberTheory/ModularForms/LevelOne.lean,Mathlib/NumberTheory/ModularForms/QExpansion.lean,Mathlib/NumberTheory/ModularForms/SlashActions.lean,Mathlib/NumberTheory/ModularForms/SlashInvariantForms.lean |
16 |
10 |
['CBirkbeck', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
1-68862 1 day ago |
1-68863 1 day ago |
0-0 0 seconds |
29560 |
loefflerd author:loefflerd |
feat(NumberTheory/ModularForms): define boundedness / vanishing at a cusp |
---
- [ ] depends on: #29327
Carved off from the larger WIP PR #26651. The changes that are new in this PR are the file `BoundedAtCusp.lean` and the two small changes in `MoebiusAction.lean` and `FunctionsBoundedAtInfty.lean`; the rest is carried over from #29327.
[](https://gitpod.io/from-referrer/)
|
t-number-theory
blocked-by-other-PR
|
392/36 |
Mathlib.lean,Mathlib/Analysis/Complex/UpperHalfPlane/FunctionsBoundedAtInfty.lean,Mathlib/Analysis/Complex/UpperHalfPlane/MoebiusAction.lean,Mathlib/LinearAlgebra/Matrix/GeneralLinearGroup/Defs.lean,Mathlib/NumberTheory/ModularForms/ArithmeticSubgroups.lean,Mathlib/NumberTheory/ModularForms/BoundedAtCusp.lean,Mathlib/NumberTheory/ModularForms/CongruenceSubgroups.lean,Mathlib/NumberTheory/ModularForms/Cusps.lean,Mathlib/NumberTheory/ModularForms/SlashInvariantForms.lean |
9 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
1-68494 1 day ago |
1-69028 1 day ago |
0-1856 30 minutes |
29204 |
ShreckYe author:ShreckYe |
feat(GroupTheory/OrderOfElement): `Pi.orderOf_eq` and its related and depended-upon theorems related to `Pi`, `minimalPeriod`, and `IsPeriodicPt` |
The need for `Pi.orderOf_eq` comes in helping prove the value of the order of a `ZMod` number when used with `ZMod.prodEquivPi`. At first I was only trying to prove `(a : (i : Fin n) → α i) : orderOf a = Finset.univ.lcm (fun i => orderOf (a i))`, but after seeing the "Corresponding `pi` lemmas" comment, I realized that this could be generalized to Pi-types (`Pi`) and also some related and dependent theorems are not implemented yet, so I went on to add and prove these referring to those similar ones for product types (`Prod`).
---
- [ ] depends on: #29530 |
t-group-theory
large-import
t-dynamics
merge-conflict
blocked-by-other-PR
|
153/10 |
Mathlib/Dynamics/PeriodicPts/Defs.lean,Mathlib/Dynamics/PeriodicPts/Lemmas.lean,Mathlib/GroupTheory/OrderOfElement.lean,Mathlib/Logic/Function/Basic.lean,Mathlib/Logic/Function/Iterate.lean |
5 |
7 |
['ShreckYe', 'github-actions', 'grunweg', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
1-61224 1 day ago |
1-61225 1 day ago |
9-60153 9 days |
29279 |
Jlh18 author:Jlh18 |
feat: free groupoid on a category, free-forgetful adjunction |
- define `CategoryTheory.Category.FreeGroupoid` in a file of the same name
- show the universal property of this construction, as the initial category localizing all maps in the category. These are the defs `of`, `lift`, and their related theorems
- Show that this construction is functorial `CategoryTheory.Category.FreeGroupoid.map`
- Convert this to a functor `CategoryTheory.Category.Grpd.free` from `Cat` to `Grpd`, and show that it is left adjoint to the forgetful functor
- `CategoryTheory.Grpd.freeForgetAdjunction`
- [ ] depends on: #29278
---
[](https://gitpod.io/from-referrer/)
|
large-import
new-contributor
blocked-by-other-PR
|
246/4 |
Mathlib.lean,Mathlib/AlgebraicTopology/FundamentalGroupoid/InducedMaps.lean,Mathlib/CategoryTheory/Category/FreeGroupoid.lean,Mathlib/CategoryTheory/Category/Grpd.lean,Mathlib/CategoryTheory/Quotient.lean |
5 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
1-49625 1 day ago |
10-31917 10 days ago |
0-1920 32 minutes |
29274 |
Jlh18 author:Jlh18 |
feat(CategoryTheory): HasLimits instance on Grpd |
- Show that the quotient of a groupoid is a groupoid in `CategoryTheory.Quotient`.
- Define the free groupoid on a category in `CategoryTheory.Category.FreeGroupoid` and hence define the free-forgetful adjunction between `Grpd` and `Cat`.
- Use the free-forgetful adjunction to show that `Grpd` has all limits in `CategoryTheory.Category.Grpd.Limit`, as a reflective subcategory of `Cat`.
- [ ] depends on: #29250[Renamings in Grpd file]
- [ ] depends on: #29278[Quotient of a groupoid is a groupoid]
- [ ] depends on: #29279[Free forgetful adjunction]
---
[](https://gitpod.io/from-referrer/)
|
large-import
new-contributor
blocked-by-other-PR
|
278/4 |
Mathlib.lean,Mathlib/AlgebraicTopology/FundamentalGroupoid/InducedMaps.lean,Mathlib/CategoryTheory/Category/FreeGroupoid.lean,Mathlib/CategoryTheory/Category/Grpd.lean,Mathlib/CategoryTheory/Groupoid/Grpd/Limit.lean,Mathlib/CategoryTheory/Quotient.lean |
6 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
1-49595 1 day ago |
10-37960 10 days ago |
0-340 5 minutes |
29561 |
j-loreaux author:j-loreaux |
feat: range of the continuous functional calculus |
---
- [ ] depends on: #29563
[](https://gitpod.io/from-referrer/)
|
t-analysis
blocked-by-other-PR
|
425/86 |
Mathlib.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Basic.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Continuity.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Instances.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Isometric.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/NonUnital.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Range.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Restrict.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Unique.lean,Mathlib/Analysis/SpecialFunctions/ContinuousFunctionalCalculus/PosPart/Basic.lean,Mathlib/Analysis/SpecialFunctions/ContinuousFunctionalCalculus/Rpow/Basic.lean,Mathlib/Topology/ContinuousMap/ContinuousMapZero.lean,Mathlib/Topology/ContinuousMap/StoneWeierstrass.lean |
13 |
3 |
['github-actions', 'j-loreaux', 'mathlib4-dependent-issues-bot'] |
nobody |
1-48736 1 day ago |
1-57301 1 day ago |
0-789 13 minutes |
29565 |
joelriou author:joelriou |
feat(CategoryTheory): dense functors |
A functor `F : C ⥤ D` is dense if any `Y : D` is a canonical colimit relatively to `F`. When `F` is full, we show that this is equivalent to saying that the restricted Yoneda functor `D ⥤ Cᵒᵖ ⥤ Type _` is fully faithful. We also show that the range of a dense functor is a strong generator.
---
- [ ] depends on: #29556
- [ ] depends on: #29519
- [ ] depends on: #29518
- [ ] depends on: #29543
[](https://gitpod.io/from-referrer/)
|
large-import
t-category-theory
blocked-by-other-PR
WIP
|
531/2 |
Mathlib.lean,Mathlib/CategoryTheory/ExtremalEpi.lean,Mathlib/CategoryTheory/Functor/Dense.lean,Mathlib/CategoryTheory/Generator/StrongGenerator.lean,Mathlib/CategoryTheory/Limits/Canonical.lean,Mathlib/CategoryTheory/Presentable/CardinalFilteredPresentation.lean |
6 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
1-47579 1 day ago |
1-47586 1 day ago |
0-1 1 second |
27268 |
wwylele author:wwylele |
feat: Hahn embedding theorem |
This proves [Hahn embedding theorem](https://en.wikipedia.org/wiki/Hahn_embedding_theorem), one among the 1000+ theorems project.
---
This is migrated from #25140 to fork, also did a general clean up so that the overall code is mathlib-ready-ish. This is still in draft state, as I split this into small PRs
- [ ] depends on: #29275
- [x] depends on: #26114
- [ ] depends on: #27043
- [x] depends on: #29421
- [x] depends on: #29423
- [x] depends on: #29451
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
blocked-by-other-PR
label:t-algebra$ |
1644/0 |
Mathlib.lean,Mathlib/Algebra/Order/Group/HahnEmbedding.lean,Mathlib/Algebra/Order/Module/HahnEmbedding.lean,Mathlib/GroupTheory/DivisibleHull.lean,docs/1000.yaml,docs/references.bib |
6 |
6 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
1-24320 1 day ago |
1-24321 1 day ago |
0-0 0 seconds |
25799 |
dagurtomas author:dagurtomas |
feat(CategoryTheory): the universal property of localized monoidal categories |
This PR provides a monoidal structure on any functor out of a localized monoidal category whose precomposition with the localization functor is monoidal
---
- [ ] depends on: #29564
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #24727.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/24727* |
t-category-theory
blocked-by-other-PR
|
729/0 |
Mathlib.lean,Mathlib/CategoryTheory/Localization/Bifunctor.lean,Mathlib/CategoryTheory/Localization/MonoidalFunctor.lean,Mathlib/CategoryTheory/Monoidal/Functor.lean,Mathlib/CategoryTheory/Monoidal/Multifunctor.lean |
5 |
7 |
['dagurtomas', 'github-actions', 'joelriou', 'mathlib4-dependent-issues-bot'] |
TwoFX assignee:TwoFX |
1-18944 1 day ago |
1-60655 1 day ago |
10-65369 10 days |
29579 |
vlad902 author:vlad902 |
feat(SimpleGraph): characterize graphs with chromatic number 1 or 2 |
- [ ] depends on: #29578 |
t-combinatorics
blocked-by-other-PR
|
53/18 |
Mathlib/Combinatorics/SimpleGraph/Basic.lean,Mathlib/Combinatorics/SimpleGraph/Coloring.lean,Mathlib/Combinatorics/SimpleGraph/ConcreteColorings.lean |
3 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
1-7061 1 day ago |
1-14621 1 day ago |
0-1604 26 minutes |
27414 |
staroperator author:staroperator |
feat(ModelTheory): Semilinear sets in `ℕ ^ k` are closed under intersection and complement |
Separated from #27100.
---
- [x] depends on: #27082
- [x] depends on: #27086
- [x] depends on: #27088
- [x] depends on: #27096
- [x] depends on: #27097
- [ ] depends on: #27342
- [x] depends on: #27957
- [ ] depends on: #28670
- [ ] depends on: #29032
---
[](https://gitpod.io/from-referrer/)
|
t-logic
merge-conflict
blocked-by-other-PR
|
1193/49 |
Mathlib.lean,Mathlib/Algebra/Group/Subgroup/Basic.lean,Mathlib/Algebra/Group/Submonoid/Operations.lean,Mathlib/Data/Set/Prod.lean,Mathlib/GroupTheory/Finiteness.lean,Mathlib/ModelTheory/Arithmetic/Presburger/Semilinear/Defs.lean,Mathlib/ModelTheory/Arithmetic/Presburger/Semilinear/Nat.lean,Mathlib/RingTheory/Finiteness/Cardinality.lean,docs/references.bib |
9 |
4 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
1-2180 1 day ago |
16-25121 16 days ago |
0-193 3 minutes |
29314 |
Louddy author:Louddy |
feat(SkewMonoidAlgebra): Lifts for skew monoid algebras |
Lemmas about different kinds of "lifts" to `SkewMonoidAlgebra` - Similar in spirit to the MonoidAlgebra.Lift file.
Co-authored-by: María Inés de Frutos Fernández <[mariaines.dff@gmail.com](mailto:mariaines.dff@gmail.com)>
---
- [ ] depends on: #29310
[](https://gitpod.io/from-referrer/)
|
blocked-by-other-PR |
293/2 |
Mathlib.lean,Mathlib/Algebra/SkewMonoidAlgebra/Basic.lean,Mathlib/Algebra/SkewMonoidAlgebra/Lift.lean |
3 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
0-79116 21 hours ago |
0-79132 21 hours ago |
0-2721 45 minutes |
26872 |
faenuccio author:faenuccio |
chore(RingTheory/Valuation/RankOne): modify the definition of Valuation.RankOne using its range rather than its codomain |
We modify the definition of `RankOne` for a valuation in terms of its `valueGroup` rather than its codomain.
Co-authored by María Inés de Frutos Fernández @mariainesdff
- [ ] depends on: #26588
- [x] depends on: #26980
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
awaiting-author
blocked-by-other-PR
label:t-algebra$ |
273/37 |
Mathlib.lean,Mathlib/Algebra/GroupWithZero/Range.lean,Mathlib/Algebra/GroupWithZero/WithZero.lean,Mathlib/Algebra/Order/GroupWithZero/Range.lean,Mathlib/Algebra/Order/GroupWithZero/WithZero.lean,Mathlib/Algebra/Order/Monoid/WithTop.lean,Mathlib/RingTheory/Valuation/Basic.lean,Mathlib/RingTheory/Valuation/RankOne.lean,Mathlib/Topology/Algebra/Valued/NormedValued.lean |
9 |
12 |
['faenuccio', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'pechersky'] |
nobody |
0-77448 21 hours ago |
0-77473 21 hours ago |
0-117 1 minute |
22059 |
grunweg author:grunweg |
feat: manifolds with smooth boundary |
Needs polish, and closing the remaining sorries (or deciding they can be postponed later).
From my bordism theory project.
---
- [x] depends on: #22070
- [x] depends on: #22128
- [x] depends on: #22131
- [x] depends on: #22082
- [x] depends on: #22113
- [x] depends on: #22105
- [x] depends on: #26099
- [x] depends on: #29589 (one fiddly sorry left)
- [ ] depends on the analogous result for direct sums, still to be written
- [ ] depends on #23040 for the mathlib-level definition of smooth immersions and embeddings
[](https://gitpod.io/from-referrer/)
|
t-differential-geometry
merge-conflict
blocked-by-other-PR
WIP
|
603/0 |
Mathlib.lean,Mathlib/Geometry/Manifold/HasSmoothBoundary.lean |
2 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
0-76323 21 hours ago |
154-72310 5 months ago |
0-0 0 seconds |
27273 |
xroblot author:xroblot |
feat(IntermediateField/LinearDisjoint): Two fields are linearly disjoint iff they are disjoint in the Galois case |
---
- [ ] depends on: #26841
[](https://gitpod.io/from-referrer/)
|
t-algebra
blocked-by-other-PR
label:t-algebra$ |
136/1 |
Mathlib/FieldTheory/Galois/Basic.lean,Mathlib/FieldTheory/IntermediateField/Basic.lean,Mathlib/FieldTheory/LinearDisjoint.lean |
3 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
0-70992 19 hours ago |
0-71023 19 hours ago |
0-1636 27 minutes |
27969 |
smmercuri author:smmercuri |
feat: collections of non-trivial and pairwise inequivalent absolute values contain values that diverge around 1 |
This PR continues the work from #22142.
Original PR: https://github.com/leanprover-community/mathlib4/pull/22142
---
- [ ] depends on: #27964 |
t-algebra
t-number-theory
blocked-by-other-PR
label:t-algebra$ |
350/40 |
Mathlib/Algebra/Order/AbsoluteValue/Basic.lean,Mathlib/Analysis/AbsoluteValue/Equivalence.lean,Mathlib/Analysis/Normed/Ring/WithAbs.lean,Mathlib/NumberTheory/Ostrowski.lean |
4 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
0-70352 19 hours ago |
38-83672 1 month ago |
0-305 5 minutes |
25794 |
dagurtomas author:dagurtomas |
feat(CategoryTheory): localization preserves braided structure |
---
- [ ] depends on: #29568
[](https://gitpod.io/from-referrer/)
---
*This PR continues the work from #24485.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/24485* |
file-removed
t-category-theory
blocked-by-other-PR
|
445/3 |
Mathlib.lean,Mathlib/CategoryTheory/Functor/CurryingThree.lean,Mathlib/CategoryTheory/Localization/Monoidal/Basic.lean,Mathlib/CategoryTheory/Localization/Monoidal/Braided.lean,Mathlib/CategoryTheory/Monoidal/Braided/Basic.lean,Mathlib/CategoryTheory/Monoidal/Braided/Multifunctor.lean,Mathlib/CategoryTheory/Sites/Monoidal.lean |
7 |
4 |
['dagurtomas', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
mattrobball assignee:mattrobball |
0-68923 19 hours ago |
1-18340 1 day ago |
45-8425 45 days |
26588 |
faenuccio author:faenuccio |
feat(Algebra/GroupWithZero/WithZero): add the multiplicative embedding with zero from the range |
We extend the embedding of the range of a `MonoidWithZeroHom` to the codomain by enriching it with the structure of an ordered, multiplicative embedding. In passing, we extend some results about the embedding of `WithZero` of the units of a group with zero, to the group itself.
Co-authored by: María Inés de Frutos Fernández @mariainesdff
---
- [ ] depends on: #29594
[](https://gitpod.io/from-referrer/)
|
t-order
t-algebra
blocked-by-other-PR
label:t-algebra$ |
132/8 |
Mathlib.lean,Mathlib/Algebra/GroupWithZero/Range.lean,Mathlib/Algebra/GroupWithZero/WithZero.lean,Mathlib/Algebra/Order/GroupWithZero/Range.lean,Mathlib/Algebra/Order/GroupWithZero/WithZero.lean,Mathlib/Algebra/Order/Monoid/WithTop.lean |
6 |
51 |
['YaelDillies', 'faenuccio', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'pechersky'] |
YaelDillies assignee:YaelDillies |
0-66545 18 hours ago |
0-71592 19 hours ago |
18-83545 18 days |
27579 |
RemyDegenne author:RemyDegenne |
feat: risk of an estimator, DeGroot statistical information, total variation distance |
This is an overview PR and will be cut into several pieces. It contains definitions and properties of:
- the risk and Bayes risk of an estimator, in general and then specialized to binary hypothesis testing
- the DeGroot statistical information between two measures, as well as a generalization for a kernel on more than two outcomes
- the total variation distance between measures, defined as a special case of the DeGroot statistical information
Co-authored-by: Lorenzo Luccioli @LorenzoLuccioli
From the TestingLowerBounds project
---
- [x] depends on: #27583
- [x] depends on: #27584
- [x] depends on: #27585
- [x] depends on: #27586
- [x] depends on: #27587
- [x] depends on: #27591
- [x] depends on: #28081
- [x] depends on: #28082
- [x] depends on: #28117
- [x] depends on: #28341
- [ ] depends on: #29137
- [ ] depends on: #29143
[](https://gitpod.io/from-referrer/)
|
t-measure-probability
merge-conflict
blocked-by-other-PR
WIP
|
1956/17 |
Mathlib.lean,Mathlib/InformationTheory/TotalVariation/Basic.lean,Mathlib/Probability/Decision/AuxLemmas.lean,Mathlib/Probability/Decision/BayesEstimator.lean,Mathlib/Probability/Decision/Binary.lean,Mathlib/Probability/Decision/BoolMeasure.lean,Mathlib/Probability/Decision/DeGrootInfo.lean,Mathlib/Probability/Decision/Risk/Basic.lean,Mathlib/Probability/Decision/Risk/Countable.lean,Mathlib/Probability/Decision/RiskIncrease.lean,Mathlib/Probability/Decision/ZeroOneLoss.lean,Mathlib/Probability/Kernel/Composition/Comp.lean,Mathlib/Probability/Kernel/Composition/MapComap.lean,Mathlib/Probability/Kernel/Defs.lean,Mathlib/Probability/Kernel/RadonNikodym.lean |
15 |
6 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
0-63942 17 hours ago |
0-63943 17 hours ago |
0-1 1 second |
29243 |
yoh-tanimoto author:yoh-tanimoto |
feat(Analysis/InnerProductSpace/Projection/Submodule): add `sup_orthogonal` for `ClosedSubmodules` |
prove that the closed submodule generated by the orthogonal complements of two submodules is the orthogonal complement of the intersection.
motivation: needed to define standard subspaces in a Hilbert space #29251
https://ems.press/content/serial-article-files/48171
- [ ] depends on: #29230 for `Lattice` `CompleteLattice`
- [ ] depends on: #29241 for the definition of `orthogonal` |
merge-conflict
blocked-by-other-PR
|
354/1 |
Mathlib/Analysis/InnerProductSpace/Orthogonal.lean,Mathlib/Analysis/InnerProductSpace/Projection/Submodule.lean,Mathlib/Topology/Algebra/Module/ClosedSubmodule.lean |
3 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
0-63058 17 hours ago |
0-63058 17 hours ago |
0-2553 42 minutes |
29251 |
yoh-tanimoto author:yoh-tanimoto |
feat(Analysis/InnerProductSpace/): define standard subspaces of a complex Hilbert space |
define standard subspaces of a complex Hilbert space: a standard subspace `S` of `H` is a closed real subspace `S` such that `S ⊓ i S = ⊥` and `S ⊔ i S = ⊤`.
prove that the symplectic complement of `S` is again a standard subspace and the double symplectic complement is itself.
motivation: one can define a closable operator `x + i y ↦ x - i y` and develop an analogue of the Tomita-Takesaki
modular theory for von Neumann algebras. By considering inclusions of standard subspaces, one can
obtain unitary representations of various Lie groups.
https://ems.press/content/serial-article-files/48171
- [ ] depends on: #29230 for `Lattice` `CompleteLattice`
- [ ] depends on: #29241 for the definition of `orthogonal`
- [ ] depends on: #29243 for `sup_orthogonal`
- [ ] depends on: #29235 for `mapEquiv` |
merge-conflict
blocked-by-other-PR
|
699/2 |
Mathlib.lean,Mathlib/Analysis/InnerProductSpace/Orthogonal.lean,Mathlib/Analysis/InnerProductSpace/Projection/Submodule.lean,Mathlib/Analysis/InnerProductSpace/StandardSubspace.lean,Mathlib/Topology/Algebra/Module/ClosedSubmodule.lean |
5 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
0-62935 17 hours ago |
0-62936 17 hours ago |
0-3098 51 minutes |
28733 |
CBirkbeck author:CBirkbeck |
E2 s transform |
---
- [ ] depends on : #29115
- [ ] depends on: #27606
- [ ] depends on" #26014
[](https://gitpod.io/from-referrer/)
|
large-import
merge-conflict
blocked-by-other-PR
|
2068/19 |
Mathlib.lean,Mathlib/Analysis/Asymptotics/Lemmas.lean,Mathlib/Analysis/Complex/Exponential.lean,Mathlib/Analysis/Complex/IntegerCompl.lean,Mathlib/Analysis/Complex/Norm.lean,Mathlib/Analysis/Complex/SummableUniformlyOn.lean,Mathlib/Analysis/Normed/Group/Basic.lean,Mathlib/Analysis/Normed/Module/Basic.lean,Mathlib/Analysis/Normed/Module/FiniteDimension.lean,Mathlib/Analysis/RCLike/Basic.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Cotangent.lean,Mathlib/NumberTheory/ArithmeticFunction.lean,Mathlib/NumberTheory/IccSums.lean,Mathlib/NumberTheory/LSeries/RiemannZeta.lean,Mathlib/NumberTheory/ModularForms/EisensteinSeries/Defs.lean,Mathlib/NumberTheory/ModularForms/EisensteinSeries/E2.lean,Mathlib/NumberTheory/ModularForms/EisensteinSeries/QExpansion.lean,Mathlib/NumberTheory/ModularForms/EisensteinSeries/Summable.lean,Mathlib/NumberTheory/TsumDivsorsAntidiagonal.lean,Mathlib/Topology/Algebra/InfiniteConditionalSum/Basic.lean,Mathlib/Topology/Algebra/InfiniteSum/Basic.lean,Mathlib/Topology/Algebra/InfiniteSum/NatInt.lean,Mathlib/Topology/Algebra/Monoid/Defs.lean,Mathlib/Topology/UniformSpace/LimUnder.lean |
24 |
n/a |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
0-61423 17 hours ago |
unknown |
unknown |
28797 |
xroblot author:xroblot |
feat(DedekindDomain/Ideal): `relNorm` of a prime ideal |
---
- [ ] depends on: #27105
- [x] depends on: #27157
- [x] depends on: #28169
- [ ] depends on: #28738
- [x] depends on: #28724
- [x] depends on: #29068
- [x] depends on: #29069
[](https://gitpod.io/from-referrer/)
|
large-import
merge-conflict
blocked-by-other-PR
|
310/4 |
Mathlib/Algebra/Group/Opposite.lean,Mathlib/Algebra/Group/Torsion.lean,Mathlib/Algebra/Ring/NonZeroDivisors.lean,Mathlib/RingTheory/Binomial.lean,Mathlib/RingTheory/DedekindDomain/Factorization.lean,Mathlib/RingTheory/DedekindDomain/Ideal/Basic.lean,Mathlib/RingTheory/DedekindDomain/Ideal/Lemmas.lean,Mathlib/RingTheory/Ideal/GoingUp.lean,Mathlib/RingTheory/Ideal/Norm/AbsNorm.lean,Mathlib/RingTheory/Ideal/Norm/RelNorm.lean,Mathlib/RingTheory/Ideal/Operations.lean,Mathlib/RingTheory/Ideal/Over.lean,Mathlib/RingTheory/UniqueFactorizationDomain/NormalizedFactors.lean |
13 |
7 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
riccardobrasca assignee:riccardobrasca |
0-58411 16 hours ago |
0-58412 16 hours ago |
0-45 45 seconds |
26858 |
Thmoas-Guan author:Thmoas-Guan |
feat(Algebra): Define the associated graded ring to filtered ring |
Define the associated graded ring to a filtered ring.
---
- [ ] depends on: #26857
[](https://gitpod.io/from-referrer/)
migrated from #20913
|
t-algebra
merge-conflict
blocked-by-other-PR
label:t-algebra$ |
436/0 |
Mathlib.lean,Mathlib/RingTheory/FilteredAlgebra/AssociatedGraded.lean |
2 |
n/a |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
0-26591 7 hours ago |
unknown |
unknown |
26859 |
Thmoas-Guan author:Thmoas-Guan |
feat(Algebra): Define associated graded algebra |
Define the associated graded algebra of a filtered algebra, constructed from a special case of associated graded ring.
---
- [ ] depends on: #26858
[](https://gitpod.io/from-referrer/)
migrated from #21806 |
t-algebra
merge-conflict
blocked-by-other-PR
label:t-algebra$ |
547/0 |
Mathlib.lean,Mathlib/RingTheory/FilteredAlgebra/AssociatedGraded.lean |
2 |
n/a |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
0-26590 7 hours ago |
unknown |
unknown |
26860 |
Thmoas-Guan author:Thmoas-Guan |
feat(Algebra): Define associated graded module |
Define the associated graded module to a filtered module.
---
- [ ] depends on: #26858
[](https://gitpod.io/from-referrer/)
migrated from #20940 |
t-algebra
merge-conflict
blocked-by-other-PR
label:t-algebra$ |
651/0 |
Mathlib.lean,Mathlib/RingTheory/FilteredAlgebra/AssociatedGraded.lean |
2 |
n/a |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
0-26588 7 hours ago |
unknown |
unknown |
26861 |
Thmoas-Guan author:Thmoas-Guan |
feat(Algebra): define filtered add group hom |
In this file we define filtered hom and the corresponding associated graded hom for abelian groups.
Co-authored-by: Huanyu Zheng @Yu-Misaka
Co-authored-by: Yi Yuan @yuanyi-350
Co-authored-by: Weichen Jiao @AlbertJ-314
---
- [ ] depends on: #26857
[](https://gitpod.io/from-referrer/)
migrated from #22632
|
t-algebra
merge-conflict
blocked-by-other-PR
label:t-algebra$ |
376/0 |
Mathlib.lean,Mathlib/RingTheory/FilteredAlgebra/AssociatedGraded.lean,Mathlib/RingTheory/FilteredAlgebra/FilteredHom.lean |
3 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
0-26587 7 hours ago |
0-26588 7 hours ago |
0-1200 20 minutes |
26862 |
Thmoas-Guan author:Thmoas-Guan |
feat(Algebra): define filtered ring homomorphism |
In this PR, we define the filtered ring morphisms on rings and prove some basic properties of
them.
Co-authored-by: Huanyu Zheng @Yu-Misaka
Co-authored-by: Yi Yuan @yuanyi-350
Co-authored-by: Weichen Jiao @AlbertJ-314
---
- [ ] depends on: #26858
- [ ] depends on: #26861
[](https://gitpod.io/from-referrer/)
migrated from #22208
|
t-algebra
merge-conflict
blocked-by-other-PR
label:t-algebra$ |
806/0 |
Mathlib.lean,Mathlib/RingTheory/FilteredAlgebra/AssociatedGraded.lean,Mathlib/RingTheory/FilteredAlgebra/FilteredHom.lean |
3 |
n/a |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
0-26586 7 hours ago |
unknown |
unknown |
26863 |
Thmoas-Guan author:Thmoas-Guan |
feat(Algebra): define filtered alghom |
In this PR, we define the filtered algebra homomorphisms on algebras and prove some basic properties of
them.
---
- [ ] depends on: #26859
- [ ] depends on: #26862
[](https://gitpod.io/from-referrer/)
migrated from #22454
|
t-algebra
merge-conflict
blocked-by-other-PR
label:t-algebra$ |
1034/0 |
Mathlib.lean,Mathlib/RingTheory/FilteredAlgebra/AssociatedGraded.lean,Mathlib/RingTheory/FilteredAlgebra/FilteredHom.lean |
3 |
n/a |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
0-26585 7 hours ago |
unknown |
unknown |
26867 |
Thmoas-Guan author:Thmoas-Guan |
feat(Algebra): filtered module hom |
In this PR we defined the filtered semi-linear map for filtered module and the associated graded module hom.
---
- [ ] depends on: #26860
- [ ] depends on: #26862
[](https://gitpod.io/from-referrer/)
migrated from #22893 |
t-algebra
merge-conflict
blocked-by-other-PR
label:t-algebra$ |
1182/0 |
Mathlib.lean,Mathlib/RingTheory/FilteredAlgebra/AssociatedGraded.lean,Mathlib/RingTheory/FilteredAlgebra/FilteredHom.lean |
3 |
n/a |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
0-26583 7 hours ago |
unknown |
unknown |
26868 |
Thmoas-Guan author:Thmoas-Guan |
feat(Algebra): associated graded exact of exact and strict |
In this file, we define the concept of exhaustive filtrations.
We also prove a AssociatedGradedRingHom sequence is exact iff each GradedPieceHom is exact.
And when a sequence is strict exact, the corresponding AssociatedGradedRingHom sequence is also exact.
Co-authored-by: Huanyu Zheng @Yu-Misaka
Co-authored-by: Yi Yuan @yuanyi-350
Co-authored-by: Weichen Jiao @AlbertJ-314
---
- [ ] depends on: #26861
[](https://gitpod.io/from-referrer/)
migrated from #22707 |
t-algebra
merge-conflict
blocked-by-other-PR
label:t-algebra$ |
532/0 |
Mathlib.lean,Mathlib/RingTheory/FilteredAlgebra/AssociatedGraded.lean,Mathlib/RingTheory/FilteredAlgebra/Exactness.lean,Mathlib/RingTheory/FilteredAlgebra/FilteredHom.lean |
4 |
n/a |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
0-26582 7 hours ago |
unknown |
unknown |
26869 |
Thmoas-Guan author:Thmoas-Guan |
feat(Algebra): exact of associated graded exact |
We proved that a chain complex is exact if its associated graded complex is exact.
Co-authored-by: Huanyu Zheng @Yu-Misaka
Co-authored-by: Yi Yuan @yuanyi-350
Co-authored-by: Weichen Jiao @AlbertJ-314
---
- [ ] depends on: #26868
[](https://gitpod.io/from-referrer/)
migrated from #22972
|
t-algebra
merge-conflict
blocked-by-other-PR
label:t-algebra$ |
723/0 |
Mathlib.lean,Mathlib/RingTheory/FilteredAlgebra/AssociatedGraded.lean,Mathlib/RingTheory/FilteredAlgebra/Exactness.lean,Mathlib/RingTheory/FilteredAlgebra/FilteredHom.lean |
4 |
n/a |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
0-26581 7 hours ago |
unknown |
unknown |
28468 |
alreadydone author:alreadydone |
feat(Algebra): ring API for `AddLocalization` |
Extract `Submonoid.IsLocalizationMap` from `LocalizationMap` and use it in `IsLocalization`.
Develop basic API for AddLocalization at a two-sided ideal; in the case of the top AddSubmonoid, show the localization has a Ring structure (Grothendieck ring).
Show that a commuative semiring with cancellative addition satisfies the strong rank condition.
---
- [x] depends on: #27842
- [x] depends on: #27862
- [ ] depends on: #29596
- [ ] depends on: #29597
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
awaiting-author
blocked-by-other-PR
label:t-algebra$ |
1000/120 |
Mathlib.lean,Mathlib/Algebra/Module/End.lean,Mathlib/Algebra/Module/LocalizedModule/IsLocalization.lean,Mathlib/Algebra/Order/Nonneg/Basic.lean,Mathlib/Algebra/Order/Nonneg/Ring.lean,Mathlib/Algebra/Ring/Invertible.lean,Mathlib/GroupTheory/MonoidLocalization/Archimedean.lean,Mathlib/GroupTheory/MonoidLocalization/Basic.lean,Mathlib/GroupTheory/MonoidLocalization/Lemmas.lean,Mathlib/GroupTheory/MonoidLocalization/MonoidWithZero.lean,Mathlib/LinearAlgebra/TensorProduct/Basic.lean,Mathlib/RingTheory/IsTensorProduct.lean,Mathlib/RingTheory/Localization/Additive.lean,Mathlib/RingTheory/Localization/Basic.lean,Mathlib/RingTheory/Localization/Defs.lean,Mathlib/RingTheory/Localization/StrongRankCondition.lean,Mathlib/RingTheory/Smooth/StandardSmooth.lean |
17 |
6 |
['alreadydone', 'chrisflav', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
chrisflav assignee:chrisflav |
0-24474 6 hours ago |
0-24475 6 hours ago |
17-3113 17 days |
28769 |
chrisflav author:chrisflav |
feat(RingTheory/Extension/Cotangent): presentation is submersive if `I/I²` has a suitable basis |
Let `P` be a presentation of an algebra with kernel `I`. We show that if `I/I²` has a basis given by the images of the relations and the module of Kaehler differentials has a basis given by the differentials of the free generators (those that don't appear in the Jacobian matrix), then `P` is submersive.
We will later deduce from this a presentation-independent characterization of standard smooth algebras.
From Pi1.
---
- [ ] depends on: #28767
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
large-import
merge-conflict
blocked-by-other-PR
|
917/561 |
Mathlib.lean,Mathlib/Algebra/Module/Submodule/Ker.lean,Mathlib/Algebra/Module/Submodule/LinearMap.lean,Mathlib/Algebra/Module/Submodule/Map.lean,Mathlib/Algebra/Module/Submodule/Range.lean,Mathlib/Data/Finsupp/Basic.lean,Mathlib/LinearAlgebra/Basis/Exact.lean,Mathlib/LinearAlgebra/Determinant.lean,Mathlib/LinearAlgebra/Finsupp/Defs.lean,Mathlib/LinearAlgebra/Finsupp/Span.lean,Mathlib/LinearAlgebra/Finsupp/Supported.lean,Mathlib/LinearAlgebra/Finsupp/VectorSpace.lean,Mathlib/LinearAlgebra/LinearIndependent/Defs.lean,Mathlib/LinearAlgebra/LinearIndependent/Lemmas.lean,Mathlib/LinearAlgebra/Projection.lean,Mathlib/RingTheory/Extension/Cotangent/Basic.lean,Mathlib/RingTheory/Extension/Cotangent/Free.lean,Mathlib/RingTheory/Extension/Presentation/Submersive.lean,Mathlib/RingTheory/Smooth/StandardSmooth.lean |
19 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
0-24349 6 hours ago |
0-24350 6 hours ago |
0-655 10 minutes |
29534 |
Thmoas-Guan author:Thmoas-Guan |
feat(Algebra): global dimension of regular local ring |
In this PR, we proved the global dimension of regular local ring is equal to its krull dimension via Auslander Buchsbaum theorem.
---
- [ ] depends on: #29557
- [ ] depends on: #26215
- [ ] depends on: #29558
[](https://gitpod.io/from-referrer/)
|
large-import
blocked-by-other-PR
WIP
|
3516/40 |
Mathlib.lean,Mathlib/Algebra/Category/Grp/Preadditive.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/LinearAlgebra/Quotient/Basic.lean,Mathlib/RingTheory/CohenMacaulay/Basic.lean,Mathlib/RingTheory/CohenMacaulay/Maximal.lean,Mathlib/RingTheory/GlobalDimension.lean,Mathlib/RingTheory/Ideal/AssociatedPrime/Localization.lean,Mathlib/RingTheory/Ideal/MinimalPrime/Localization.lean,Mathlib/RingTheory/Jacobson/Ideal.lean,Mathlib/RingTheory/KrullDimension/Module.lean,Mathlib/RingTheory/KrullDimension/Regular.lean,Mathlib/RingTheory/LocalRing/MaximalIdeal/Basic.lean,Mathlib/RingTheory/Nakayama.lean,Mathlib/RingTheory/Regular/AuslanderBuchsbaum.lean,Mathlib/RingTheory/Regular/Category.lean,Mathlib/RingTheory/Regular/Depth.lean,Mathlib/RingTheory/Regular/Ischebeck.lean,Mathlib/RingTheory/RegularLocalRing/Basic.lean,Mathlib/RingTheory/RegularLocalRing/Defs.lean,Mathlib/RingTheory/RegularLocalRing/GlobalDimension.lean,Mathlib/RingTheory/Support.lean |
22 |
n/a |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
0-17638 4 hours ago |
unknown |
unknown |