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 |
| 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 |
492-67 1 year ago |
520-59147 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 |
492-66 1 year ago |
unknown |
unknown |
| 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 |
492-63 1 year ago |
686-41309 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 |
492-63 1 year ago |
697-74494 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 |
476-78854 1 year ago |
476-78854 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 |
476-76002 1 year ago |
476-76002 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 |
476-74316 1 year ago |
476-74316 1 year ago |
50-50444 50 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 |
472-63106 1 year ago |
476-76032 1 year ago |
16-44803 16 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 |
462-45648 1 year ago |
462-45648 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 |
459-75653 1 year ago |
459-75653 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 |
459-38598 1 year ago |
490-84257 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 |
458-55391 1 year ago |
463-2500 1 year ago |
1-43047 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 |
451-62257 1 year ago |
452-21105 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 |
450-54249 1 year ago |
602-66987 1 year ago |
55-82183 55 days |
| 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 |
410-85630 1 year ago |
652-77699 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 |
408-57600 1 year ago |
408-57600 1 year ago |
31-44440 31 days |
| 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 |
330-55686 10 months ago |
330-55686 10 months ago |
4-64422 4 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 |
318-82135 10 months ago |
318-82135 10 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 |
318-68900 10 months ago |
319-69853 10 months ago |
2-77310 2 days |
| 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 |
304-53302 10 months ago |
304-53305 10 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 |
301-79262 9 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 |
301-73352 9 months ago |
301-73352 9 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 |
301-73121 9 months ago |
301-73121 9 months ago |
0-0 0 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 |
288-33742 9 months ago |
288-33742 9 months ago |
13-33168 13 days |
| 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 |
275-46659 9 months ago |
311-50436 10 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 |
272-2418 8 months ago |
273-58104 8 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 |
269-42491 8 months ago |
269-65235 8 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 |
268-46999 8 months ago |
268-48939 8 months ago |
0-0 0 seconds |
| 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 |
261-80597 8 months ago |
261-80752 8 months ago |
0-1 1 second |
| 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 |
258-83743 8 months ago |
258-83743 8 months ago |
0-68906 19 hours |
| 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 |
241-78842 7 months ago |
242-65141 7 months ago |
4-80306 4 days |
| 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 |
235-34050 7 months ago |
235-72002 7 months ago |
0-1 1 second |
| 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 |
233-57060 7 months ago |
233-61860 7 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 |
233-38014 7 months ago |
507-55894 1 year ago |
57-4216 57 days |
| 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 |
231-41458 7 months ago |
360-63031 11 months ago |
370-50661 370 days |
| 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 |
226-60291 7 months ago |
226-60291 7 months ago |
0-2221 37 minutes |
| 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 |
216-6637 7 months ago |
256-46346 8 months ago |
2-24624 2 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 |
216-2482 7 months ago |
216-2482 7 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 |
216-1512 7 months ago |
216-1512 7 months ago |
0-0 0 seconds |
| 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 |
214-71696 7 months ago |
221-13848 7 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 |
214-42764 7 months ago |
214-77378 7 months ago |
0-0 0 seconds |
| 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 |
212-36647 6 months ago |
212-36647 6 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 |
211-45421 6 months ago |
211-45421 6 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 |
210-35859 6 months ago |
210-35859 6 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 |
210-35625 6 months ago |
210-35625 6 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 |
210-33002 6 months ago |
210-33002 6 months ago |
20-83091 20 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 |
209-55196 6 months ago |
209-55196 6 months ago |
46-55730 46 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 |
207-80740 6 months ago |
207-80740 6 months ago |
27-52316 27 days |
| 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 |
204-68273 6 months ago |
213-48211 6 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 |
202-67417 6 months ago |
202-68867 6 months ago |
202-68913 202 days |
| 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 |
186-6744 6 months ago |
186-6744 6 months ago |
48-7769 48 days |
| 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 |
182-69648 5 months ago |
182-70538 5 months ago |
0-11212 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 |
180-44763 5 months ago |
180-44764 5 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 |
179-77871 5 months ago |
180-20407 5 months ago |
0-0 0 seconds |
| 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 |
177-26846 5 months ago |
177-28937 5 months ago |
53-20069 53 days |
| 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 |
173-55546 5 months ago |
173-55572 5 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 |
172-61336 5 months ago |
172-61339 5 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 |
172-59480 5 months ago |
172-59568 5 months ago |
0-0 0 seconds |
| 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 |
170-47347 5 months ago |
170-47347 5 months ago |
2-11832 2 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 |
167-39180 5 months ago |
167-39180 5 months ago |
0-1331 22 minutes |
| 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 |
165-35959 5 months ago |
303-6273 10 months ago |
0-0 0 seconds |
| 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 |
164-33976 5 months ago |
164-34065 5 months ago |
0-0 0 seconds |
| 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 |
156-84377 5 months ago |
156-84377 5 months ago |
14-37502 14 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 |
152-69433 4 months ago |
152-69468 4 months ago |
185-56732 185 days |
| 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 |
149-83960 4 months ago |
150-47511 4 months ago |
0-0 0 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 |
146-62617 4 months ago |
146-64039 4 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 |
144-43050 4 months ago |
144-55534 4 months ago |
0-13398 3 hours |
| 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 |
140-77096 4 months ago |
283-76601 9 months ago |
41-32344 41 days |
| 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 |
136-21221 4 months ago |
136-41546 4 months ago |
0-0 0 seconds |
| 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 |
133-58329 4 months ago |
133-58667 4 months ago |
0-29 29 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 |
131-75562 4 months ago |
131-75633 4 months ago |
0-2 2 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 |
126-43778 4 months ago |
127-77026 4 months ago |
0-0 0 seconds |
| 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 |
126-69975 4 months ago |
126-69975 4 months ago |
0-52136 14 hours |
| 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 |
125-73756 4 months ago |
125-74954 4 months ago |
0-14 14 seconds |
| 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 |
125-55238 4 months ago |
125-58320 4 months ago |
0-8982 2 hours |
| 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 |
125-17766 4 months ago |
144-35449 4 months 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 |
124-58890 4 months ago |
172-59776 5 months ago |
0-8 8 seconds |
| 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 |
124-21257 4 months ago |
124-68157 4 months ago |
15-64386 15 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 |
122-79314 4 months ago |
122-79314 4 months 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 |
122-79252 4 months ago |
unknown |
unknown |
| 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 |
118-39664 3 months ago |
118-83483 3 months ago |
0-85904 23 hours |
| 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 |
117-25099 3 months ago |
117-25109 3 months ago |
0-0 0 seconds |
| 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 |
115-58160 3 months ago |
115-58196 3 months ago |
0-1886 31 minutes |
| 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 |
115-13987 3 months ago |
115-28067 3 months ago |
25-83942 25 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 |
113-76511 3 months ago |
113-76714 3 months ago |
4-24257 4 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 |
109-42138 3 months ago |
122-79423 4 months ago |
5-42837 5 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 |
108-75139 3 months ago |
505-9453 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 |
108-74410 3 months ago |
108-74429 3 months ago |
0-0 0 seconds |
| 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 |
107-80792 3 months ago |
107-83311 3 months ago |
0-22 22 seconds |
| 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 |
107-43651 3 months ago |
107-43651 3 months ago |
19-20394 19 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 |
106-86315 3 months ago |
106-86315 3 months 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 |
106-66676 3 months ago |
106-66676 3 months ago |
0-24645 6 hours |
| 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 |
105-61200 3 months ago |
105-61200 3 months ago |
64-11252 64 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 |
103-58819 3 months ago |
127-36716 4 months ago |
0-533 8 minutes |
| 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 |
103-58464 3 months ago |
103-58506 3 months ago |
72-55831 72 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 |
103-41831 3 months ago |
103-41881 3 months ago |
0-0 0 seconds |
| 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 |
100-83756 3 months ago |
122-65733 4 months ago |
86-39206 86 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 |
99-8588 3 months ago |
99-8614 3 months ago |
0-0 0 seconds |
| 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 |
97-83676 3 months ago |
97-83798 3 months ago |
66-73556 66 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 |
95-44028 3 months ago |
115-5294 3 months ago |
0-0 0 seconds |
| 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 |
92-58427 3 months ago |
94-15897 3 months ago |
94-15928 94 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 |
92-32103 3 months ago |
148-67177 4 months ago |
148-67221 148 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 |
91-3978 3 months ago |
91-3978 3 months ago |
18-47707 18 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 |
89-63282 2 months ago |
113-54810 3 months ago |
55-10605 55 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 |
87-66169 2 months ago |
87-66209 2 months ago |
0-42619 11 hours |
| 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 |
87-30187 2 months ago |
87-61290 2 months ago |
73-43225 73 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 |
86-44942 2 months ago |
86-85377 2 months ago |
27-76128 27 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 |
85-23566 2 months ago |
85-24246 2 months ago |
0-1 1 second |
| 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 |
84-60811 2 months ago |
175-68644 5 months ago |
0-11893 3 hours |
| 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 |
82-79255 2 months ago |
82-79325 2 months ago |
82-79313 82 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 |
79-43793 2 months ago |
99-6730 3 months ago |
99-76654 99 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', 'fpvandoorn', 'github-actions', 'madvorak', 'vihdzp'] |
fpvandoorn assignee:fpvandoorn |
78-80526 2 months ago |
104-81311 3 months ago |
17-70200 17 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
awaiting-author
|
8/2 |
Mathlib/Order/SuccPred/Basic.lean |
1 |
3 |
['YaelDillies', 'github-actions', 'plp127', 'vihdzp'] |
bryangingechen assignee:bryangingechen |
76-38141 2 months ago |
76-38141 2 months ago |
44-13238 44 days |
| 29870 |
mckoen author:mckoen |
feat(CategoryTheory/Adhesive): subobjects in adhesive categories have binary coproducts |
A formalization of Theorem 5.1 in https://www.ioc.ee/~pawel/papers/adhesivejournal.pdf. Given `A B Z : C` with `C` adhesive, and `a : A ⟶ Z`, ` b : B ⟶ Z` monomorphisms, then `pushout.desc a b pullback.condition` is also a monomorphism. This result will be useful in showing that the pushout-product of monomorphisms is also a monomorphism.
---
[](https://gitpod.io/from-referrer/)
|
t-category-theory
WIP
|
118/0 |
Mathlib/CategoryTheory/Adhesive.lean |
1 |
1 |
['github-actions'] |
nobody |
74-33545 2 months ago |
74-33592 2 months ago |
0-9 9 seconds |
| 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
|
10/0 |
Mathlib/Geometry/Euclidean/Triangle.lean,docs/1000.yaml |
2 |
16 |
['FrankieNC', 'JovanGerb', 'dsfxcimk', 'github-actions', 'grunweg', 'mathlib4-merge-conflict-bot', 'themathqueen'] |
nobody |
72-55898 2 months ago |
86-68765 2 months ago |
28-57160 28 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
awaiting-author
|
383/0 |
Mathlib/Analysis/Complex/Residue/Basic.lean |
1 |
17 |
['Periecle', 'github-actions', 'hrmacbeth', 'llllvvuu', 'loefflerd'] |
nobody |
71-64289 2 months ago |
82-66392 2 months ago |
1-5255 1 day |
| 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
awaiting-author
|
7/4 |
Mathlib/Data/Finsupp/Pointwise.lean |
1 |
8 |
['Paul-Lez', 'eric-wieser', 'github-actions', 'kckennylau', 'pechersky'] |
pechersky assignee:pechersky |
66-22877 2 months ago |
66-23116 2 months ago |
168-19511 168 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
awaiting-author
|
360/0 |
MathlibTest/Junk.lean |
1 |
17 |
['NotWearingPants', 'Timeroot', 'bryangingechen', 'github-actions', 'leanprover-community-bot-assistant', 'madvorak', 'pechersky', 'vihdzp'] |
pechersky assignee:pechersky |
66-21367 2 months ago |
66-21367 2 months ago |
96-70055 96 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
awaiting-author
|
2/3 |
Mathlib/Data/ZMod/Defs.lean |
1 |
2 |
['github-actions', 'jcommelin'] |
pechersky assignee:pechersky |
66-20586 2 months ago |
66-20586 2 months ago |
46-561 46 days |
| 30142 |
shalliso author:shalliso |
feat(Topology/Baire): define IsNonMeagre |
non-meagre sets (also known as "of the second category") are worthy of their own definition and API. This was useful to me for formalizing a result of "automatic continuity", that is, a Baire-measurable homomorphism between Polish groups must be continuous. Simply working with the negation of IsMeagre quickly became cumbersome, and non-meagre sets have an important role in the study of Polish (e.g. locally compact) groups.
From https://github.com/shalliso/automatic_continuity
[ ] depends on: #30141
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-topology
|
83/1 |
Mathlib/Topology/Baire/NonMeagre.lean,Mathlib/Topology/GDelta/Basic.lean |
2 |
1 |
['github-actions'] |
nobody |
63-36420 2 months ago |
63-36422 2 months ago |
63-36461 63 days |
| 30079 |
dagurtomas author:dagurtomas |
feat(CategoryTheory): IsSheafFor as a multiequalizer condition |
---
[](https://gitpod.io/from-referrer/)
|
t-category-theory
WIP
|
112/0 |
Mathlib/CategoryTheory/Sites/Multifork.lean |
1 |
3 |
['chrisflav', 'github-actions', 'joelriou'] |
nobody |
63-32584 2 months ago |
66-11332 2 months ago |
0-1 1 second |
| 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$ |
101/125 |
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 |
11 |
['fpvandoorn', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-merge-conflict-bot'] |
nobody |
61-81530 2 months ago |
61-81564 2 months ago |
0-17 17 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
awaiting-author
|
196/0 |
Archive.lean,Archive/Imo/Imo1975Q3.lean |
2 |
36 |
['Antidite', 'LLaurance', 'github-actions', 'jsm28'] |
jsm28 assignee:jsm28 |
61-45079 2 months ago |
61-45079 2 months ago |
46-38383 46 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
awaiting-author
|
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 |
6 |
['faenuccio', 'github-actions', 'mathlib4-merge-conflict-bot', 'riccardobrasca'] |
riccardobrasca assignee:riccardobrasca |
60-31422 1 month ago |
60-31422 1 month ago |
79-37394 79 days |
| 30135 |
erdOne author:erdOne |
feat(RingTheory): `ValuativeRel` on subrings |
---
@pechersky do we want this?
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
awaiting-author
|
19/0 |
Mathlib/RingTheory/Valuation/ValuativeRel/Basic.lean |
1 |
5 |
['erdOne', 'github-actions', 'pechersky'] |
nobody |
59-58760 1 month ago |
60-31452 1 month ago |
3-20137 3 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
awaiting-author
|
95/0 |
Mathlib/Data/Nat/Factors.lean |
1 |
11 |
['b-mehta', 'github-actions', 'grunweg', 'plp127'] |
b-mehta assignee:b-mehta |
53-71262 1 month ago |
54-12075 1 month ago |
111-15071 111 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
help-wanted
|
24/0 |
Mathlib/Topology/Order/LiminfLimsup.lean |
1 |
4 |
['b-mehta', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
52-13720 1 month ago |
52-13799 1 month ago |
0-6 6 seconds |
| 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
awaiting-author
|
19/0 |
Mathlib/Data/Fintype/Quotient.lean |
1 |
12 |
['github-actions', 'kckennylau', 'pechersky', 'tristan-f-r', 'vihdzp'] |
pechersky assignee:pechersky |
50-12127 1 month ago |
50-12127 1 month ago |
88-10285 88 days |
| 30119 |
Ruben-VandeVelde author:Ruben-VandeVelde |
feat: WithTop/Bot.mapD |
To replace Option.elim; working towards #27918
---
[](https://gitpod.io/from-referrer/)
|
t-order
awaiting-author
|
32/4 |
Mathlib/Order/Hom/WithTopBot.lean,Mathlib/Order/WithBot.lean |
2 |
4 |
['JovanGerb', 'YaelDillies', 'github-actions'] |
YaelDillies assignee:YaelDillies |
49-66170 1 month ago |
51-82708 1 month ago |
12-3204 12 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
|
1932/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 |
3 |
['JovanGerb', 'github-actions', 'lecopivo'] |
nobody |
49-58521 1 month ago |
87-72354 2 months ago |
0-11559 3 hours |
| 29855 |
eric-wieser author:eric-wieser |
chore(Data/Finset/Sort): lemmas about `0 : Fin _` and `Fin.last _` |
We already had these for `⟨0, ⋯⟩` and `⟨k - 1, ⋯⟩`.
Moves:
- `Finset.orderEmbOfFin_zero` -> `Finset.orderEmbOfFin_mk_zero`
- `Finset.orderEmbOfFin_last` -> `Finset.orderEmbOfFin_mk_last`
---
[](https://gitpod.io/from-referrer/)
|
t-data
t-order
easy
delegated
|
17/7 |
Mathlib/Combinatorics/Enumerative/Composition.lean,Mathlib/Data/Finset/Sort.lean |
2 |
4 |
['eric-wieser', 'github-actions', 'mathlib-bors', 'ocfnash'] |
nobody |
49-45752 1 month ago |
70-77842 2 months ago |
3-79002 3 days |
| 29634 |
YaelDillies author:YaelDillies |
feat: missing instance `NonUnitalCommSemiring R → NonUnitalNonAssocCommSemiring R` |
For some reason, this causes elaboration issues.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
awaiting-CI
help-wanted
label:t-algebra$ |
16/7 |
Mathlib/Algebra/Ring/Defs.lean,Mathlib/RingTheory/Coalgebra/Basic.lean,Mathlib/RingTheory/Coalgebra/Hom.lean,Mathlib/Tactic/Ring/Basic.lean |
4 |
7 |
['YaelDillies', 'alreadydone', 'github-actions', 'riccardobrasca'] |
nobody |
48-58817 1 month ago |
81-81034 2 months ago |
0-19 19 seconds |
| 30460 |
janithamalith author:janithamalith |
feat(Nat): add lemma nat_card_orbit_mul_card_stabilizer_eq_card_group |
Added a lemma `nat_card_orbit_mul_card_stabilizer_eq_card_group` which is the Nat.card version of MulAction.card_orbit_mul_card_stabilizer_eq_card_group
---
[](https://gitpod.io/from-referrer/)
|
t-group-theory
new-contributor
awaiting-author
|
6/0 |
Mathlib/GroupTheory/GroupAction/CardCommute.lean |
1 |
17 |
['github-actions', 'kckennylau', 'plp127', 'tb65536'] |
tb65536 assignee:tb65536 |
45-64634 1 month ago |
45-64634 1 month ago |
8-8414 8 days |
| 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`.
---
- [x] 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
t-category-theory
delegated
|
182/2 |
Mathlib/AlgebraicTopology/SimplexCategory/GeneratorsRelations/NormalForms.lean |
1 |
6 |
['github-actions', 'joelriou', 'mathlib-bors', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
44-65422 1 month ago |
45-57138 1 month ago |
0-22513 6 hours |
| 30209 |
Ruben-VandeVelde author:Ruben-VandeVelde |
feat: some TwoSidedIdeal.span lemmas |
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
FLT
awaiting-author
|
16/0 |
Mathlib/RingTheory/TwoSidedIdeal/Operations.lean |
1 |
2 |
['erdOne', 'github-actions'] |
erdOne assignee:erdOne |
44-35928 1 month ago |
44-35928 1 month ago |
17-9153 17 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
awaiting-author
|
16/0 |
Mathlib/Combinatorics/SimpleGraph/Trails.lean |
1 |
6 |
['IvanRenison', 'github-actions', 'vlad902'] |
kmill assignee:kmill |
44-28166 1 month ago |
44-28166 1 month ago |
148-3717 148 days |
| 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
awaiting-author
|
1310/0 |
Archive.lean,Archive/Imo/Imo2025Q1.lean |
2 |
8 |
['github-actions', 'kim-em', 'mathlib4-merge-conflict-bot', 'zhuyizheng'] |
dwrensha assignee:dwrensha |
43-63976 1 month ago |
44-28680 1 month ago |
65-5080 65 days |
| 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
awaiting-author
|
48/2 |
Mathlib/CategoryTheory/Adjunction/PartialAdjoint.lean |
1 |
1 |
['github-actions'] |
nobody |
43-60402 1 month ago |
43-60402 1 month ago |
98-12071 98 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 |
7 |
['YaelDillies', 'alreadydone', 'github-actions', 'kckennylau'] |
nobody |
43-53955 1 month ago |
126-4666 4 months ago |
15-75841 15 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
please-adopt
|
387/19 |
Mathlib/Tactic/Linter/DirectoryDependency.lean,scripts/README.md,scripts/forbiddenDirs.json |
3 |
4 |
['Vierkantor', 'github-actions', 'grunweg', 'mathlib4-merge-conflict-bot'] |
nobody |
42-70366 1 month ago |
42-70399 1 month ago |
126-49390 126 days |
| 30828 |
DeVilhena-Paulo author:DeVilhena-Paulo |
feat: implementation of `Finmap.merge` |
The main contribution of this pull request is the implementation of a `merge` function for finite maps (`Finmap`). The construction relies on the definition of a `merge` function for association lists (`AList`).
There is also a side (unrelated) contribution on `Mathlib/Data/List/Permutation.lean`: the addition of a theorem about the permutation of a list with a head element (that is, a list of the form `a :: l`).
---
[](https://gitpod.io/from-referrer/)
|
t-data
new-contributor
|
449/3 |
Mathlib/Data/Finmap.lean,Mathlib/Data/List/AList.lean,Mathlib/Data/List/Permutation.lean,Mathlib/Data/List/Sigma.lean |
4 |
1 |
['github-actions'] |
nobody |
42-51598 1 month ago |
42-51677 1 month ago |
42-51725 42 days |
| 30902 |
adomani author:adomani |
chore: longLine warnings happen starting at the 101st character |
Right now, the longLine linter warning spans the whole line. This PR changes the behaviour and the warning only covers the characters exceeding the 100 character limit.
Previous discussion:
[#general > error lens in lean4 @ 💬](https://leanprover.zulipchat.com/#narrow/channel/113488-general/topic/error.20lens.20in.20lean4/near/547074537)
Specific thread:
[#mathlib4 > Restrict longLine warning to exceeding characters @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Restrict.20longLine.20warning.20to.20exceeding.20characters/near/547081669)
---
[](https://gitpod.io/from-referrer/)
|
awaiting-zulip
t-linter
|
1/1 |
Mathlib/Tactic/Linter/Style.lean |
1 |
1 |
['github-actions'] |
nobody |
40-41327 1 month ago |
40-41584 1 month ago |
0-132 2 minutes |
| 30914 |
eric-wieser author:eric-wieser |
feat(Data/Set/NAry): lemmas for `diff` |
---
[](https://gitpod.io/from-referrer/)
|
t-data
t-order
delegated
|
10/0 |
Mathlib/Data/Set/NAry.lean |
1 |
2 |
['github-actions', 'grunweg', 'mathlib-bors'] |
nobody |
39-55510 1 month ago |
39-55510 1 month ago |
0-56942 15 hours |
| 30378 |
mans0954 author:mans0954 |
refactor(Order/Hom/Lattice): Use default `initialize_simps_projections` configuration for `LatticeHom`. |
Use default `initialize_simps_projections` configuration for `LatticeHom`.
I'm not sure what was originally intended by the TODO, but this appears to work.
---
[](https://gitpod.io/from-referrer/)
|
t-order
awaiting-author
|
4/7 |
Mathlib/Order/Hom/Lattice.lean,Mathlib/Order/Hom/WithTopBot.lean |
2 |
3 |
['bryangingechen', 'fpvandoorn', 'github-actions'] |
bryangingechen assignee:bryangingechen |
37-71024 1 month ago |
38-44888 1 month ago |
18-11603 18 days |
| 30667 |
FrederickPu author:FrederickPu |
Subgroup mul |
Title:
Algebra: pointwise products for subgroups
Description:
showed the point-wise product of disjoint subgroups is equivalent to their Cartesian product
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-algebra
awaiting-author
label:t-algebra$ |
47/0 |
Mathlib/Algebra/Group/Subgroup/Pointwise.lean |
1 |
10 |
['FrederickPu', 'eric-wieser', 'github-actions', 'plp127', 'tb65536'] |
nobody |
37-64596 1 month ago |
46-54630 1 month ago |
0-46291 12 hours |
| 31013 |
vihdzp author:vihdzp |
chore: deprecate `AsLinearOrder` |
This goes back to Lean 3 (https://github.com/leanprover-community/mathlib3/pull/4037). It was used to prove two results about "linearly ordered lattices" [`le_sup_iff`](https://leanprover-community.github.io/mathlib4_docs/Mathlib/Order/Lattice.html#le_sup_iff) and [`inf_le_iff`](https://leanprover-community.github.io/mathlib4_docs/Mathlib/Order/Lattice.html#inf_le_iff) which have long since been turned into theorems on linear orders. The proper way to deal with a totally ordered partial order is to just write a `LinearOrder` instance, so there is no need for this.
---
See some brief [Zulip](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/AsLinearOrder/near/547525036) discussion.
[](https://gitpod.io/from-referrer/)
|
t-order
awaiting-author
|
7/5 |
Mathlib/Order/Basic.lean |
1 |
2 |
['github-actions', 'j-loreaux', 'urkud'] |
nobody |
37-37497 1 month ago |
37-56264 1 month ago |
0-3299 54 minutes |
| 30575 |
urkud author:urkud |
feat: lemmas about `_ • _` on Filters |
as well as `Set.Finite.f?derivWithin_eq`.
I wrote these lemmas for #24019, but the final version of that PR doesn't need them. I moved them here so that I don't forget to prepare a non-draft PR with these lemmas.
---
[](https://gitpod.io/from-referrer/)
|
t-topology |
51/0 |
Mathlib/Topology/TODO.lean |
1 |
3 |
['github-actions', 'plp127', 'urkud'] |
nobody |
37-54933 1 month ago |
50-74597 1 month ago |
0-0 0 seconds |
| 30975 |
mariainesdff author:mariainesdff |
feat(Data/Finsupp/Defs): add Finsupp.restrict |
Co-authored by: @AntoineChambert-Loir
---
[](https://gitpod.io/from-referrer/)
|
t-data
awaiting-author
|
49/0 |
Mathlib/Data/Finsupp/Defs.lean |
1 |
n/a |
['ADedecker', 'github-actions'] |
nobody |
36-59733 1 month ago |
unknown |
unknown |
| 30408 |
kckennylau author:kckennylau |
feat(RingTheory): more algebra instances for HomogeneousLocalization and linear constructors |
This PR introduces the instance `Algebra R₀ (HomogeneousLocalization 𝒜 x)` as well as two linear constructors `mkₗ` and `Away.mkₗ` that fix the denominator.
Zulip discussion: [#mathlib4 > Some algebra instance for graded algebra and homog loc](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Some.20algebra.20instance.20for.20graded.20algebra.20and.20homog.20loc/with/544178649)
---
Split from #26061.
[](https://gitpod.io/from-referrer/)
|
t-ring-theory |
65/20 |
Mathlib/RingTheory/GradedAlgebra/HomogeneousLocalization.lean |
1 |
5 |
['github-actions', 'mariainesdff'] |
mariainesdff assignee:mariainesdff |
34-30747 1 month ago |
34-30804 1 month ago |
52-16792 52 days |
| 30631 |
ADedecker author:ADedecker |
refactor: evaluation of power series in semirings |
---
[](https://gitpod.io/from-referrer/)
|
|
665/71 |
Mathlib/Algebra/Module/Congruence/Defs.lean,Mathlib/RingTheory/MvPowerSeries/EvaluationSemi.lean,Mathlib/Topology/Algebra/LinearTopology.lean,Mathlib/Topology/Algebra/LinearUniformity.lean,Mathlib/Topology/Algebra/TopologicallyNilpotent.lean |
5 |
1 |
['github-actions'] |
nobody |
33-63095 1 month ago |
48-73943 1 month 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
awaiting-author
|
6/0 |
Mathlib/Analysis/InnerProductSpace/PiL2.lean |
1 |
7 |
['Ruben-VandeVelde', 'Sebi-Kumar', 'github-actions', 'kckennylau'] |
urkud assignee:urkud |
31-80494 1 month ago |
31-80494 1 month ago |
82-22614 82 days |
| 29871 |
zach1502 author:zach1502 |
feat(Matrix/Transvection): Gauss pivot determinant identity and pivot preservation |
This PR adds two lemmas formalizing standard Gaussian pivot identities:
* `Matrix.Transvection.listTransvecCol_mul_mul_listTransvecRow_pivot`:
After applying the canonical left/right transvection products that clear the last column and row,
the pivot (bottom-right) entry of a matrix is unchanged.
Marked `@[simp]`.
* `Matrix.Transvection.det_eq_detTopLeft_mul_pivot`:
If the pivot entry is nonzero, then the determinant of the matrix factors as
the determinant of the top-left block times the pivot entry, after performing
the canonical transvections.
This is the usual Gauss–pivot determinant identity.
* Added simple usage tests in `MathlibTest/matrix.lean` to check that the new lemmas
are usable by `simp`/`simpa`.
---
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-algebra
awaiting-author
label:t-algebra$ |
94/0 |
Mathlib/LinearAlgebra/Matrix/Transvection.lean,MathlibTest/matrix.lean |
2 |
3 |
['github-actions', 'riccardobrasca', 'zach1502'] |
nobody |
31-75288 1 month ago |
31-75288 1 month ago |
42-32522 42 days |
| 30109 |
scholzhannah author:scholzhannah |
feat: the subcomplexes of a (relative classical) CW complex form a completely distributive lattice |
In this PR we prove that the space of subcomplexes `Subcomplex C` of a (relative classical) CW complex `C` is a `CompletelyDistribLattice`.
---
[](https://gitpod.io/from-referrer/)
|
t-topology
awaiting-author
|
368/1 |
Mathlib/Order/Lattice.lean,Mathlib/Topology/CWComplex/Classical/Subcomplex.lean |
2 |
19 |
['ADedecker', 'github-actions', 'scholzhannah'] |
nobody |
31-64269 1 month ago |
31-64269 1 month ago |
6-69887 6 days |
| 30158 |
nicolaviolette author:nicolaviolette |
feat: combinatorics simplegraph basic |
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-combinatorics
awaiting-author
|
9/4 |
Mathlib/Combinatorics/SimpleGraph/Basic.lean |
1 |
3 |
['b-mehta', 'github-actions'] |
b-mehta assignee:b-mehta |
31-8418 1 month ago |
31-8418 1 month ago |
31-69826 31 days |
| 30431 |
kckennylau author:kckennylau |
feat(RingTheory): a homogeneous submodule is the span of its homogeneous elements |
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory |
22/0 |
Mathlib/RingTheory/GradedAlgebra/Homogeneous/Ideal.lean,Mathlib/RingTheory/GradedAlgebra/Homogeneous/Submodule.lean |
2 |
7 |
['github-actions', 'kckennylau', 'mariainesdff'] |
mariainesdff assignee:mariainesdff |
30-70927 1 month ago |
31-49486 1 month ago |
54-81933 54 days |
| 27229 |
WilliamCoram author:WilliamCoram |
feat(GroupTheory/DoubleCoset): multiple lemmas |
From FLT
---
[](https://gitpod.io/from-referrer/)
|
t-group-theory
FLT
new-contributor
|
88/0 |
Mathlib/GroupTheory/DoubleCoset.lean |
1 |
31 |
['Ruben-VandeVelde', 'WilliamCoram', 'github-actions', 'kim-em', 'mariainesdff', 'mathlib4-merge-conflict-bot'] |
mariainesdff assignee:mariainesdff |
30-63317 1 month ago |
31-54261 1 month ago |
124-6401 124 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
awaiting-author
|
44/0 |
Mathlib/MeasureTheory/Constructions/UnitInterval.lean,Mathlib/Topology/UnitInterval.lean |
2 |
8 |
['gaetanserre', 'github-actions', 'j-loreaux', 'mathlib4-merge-conflict-bot', 'ocfnash'] |
j-loreaux assignee:j-loreaux |
30-62772 1 month ago |
30-63247 1 month ago |
97-76852 97 days |
| 30608 |
grunweg author:grunweg |
feat: another lemma about derivatives of parametric integrals |
On the path towards proving that integrating smooth functions is smooth.
From the sphere-eversion project; I am just upstreaming this.
---
[](https://gitpod.io/from-referrer/)
|
t-analysis
awaiting-author
|
125/0 |
Mathlib/Analysis/Calculus/ParametricIntegral.lean |
1 |
7 |
['Ruben-VandeVelde', 'github-actions', 'j-loreaux'] |
j-loreaux assignee:j-loreaux |
30-61958 1 month ago |
30-61958 1 month ago |
18-81847 18 days |
| 30612 |
grunweg author:grunweg |
feat: add ContDiff.lipschitzOnWith |
A C¹ function is Lipschitz on each convex compact set. From sphere-eversion.
Re-done version of https://github.com/leanprover-community/mathlib4/pull/12673.
---
Help completing the last sorries is welcome!
[](https://gitpod.io/from-referrer/)
|
t-analysis
awaiting-author
|
82/10 |
Mathlib/Analysis/Calculus/ContDiff/RCLike.lean |
1 |
6 |
['github-actions', 'grunweg', 'ocfnash', 'peabrainiac'] |
ocfnash assignee:ocfnash |
30-55438 1 month ago |
30-55460 1 month ago |
0-1970 32 minutes |
| 30560 |
dwrensha author:dwrensha |
fix(LinearAlgebra/Alternating/Basic): avoid deep recursion in MultilinearMap.alternatization |
Makes `MultilinearMap.alternatization` an `irreducible_def` to avoid errors
about deep recursion.
This is an update of #15045 according to the suggestions in [this zulip thread](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/kernel.20deep.20recursion.20detected/near/454301820).
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
awaiting-author
label:t-algebra$ |
36/9 |
Mathlib/LinearAlgebra/Alternating/Basic.lean,Mathlib/LinearAlgebra/Matrix/SpecialLinearGroup.lean,MathlibTest/DetOne.lean |
3 |
6 |
['dagurtomas', 'dwrensha', 'eric-wieser', 'github-actions'] |
dagurtomas assignee:dagurtomas |
29-54558 29 days ago |
29-54558 29 days ago |
21-72141 21 days |
| 31226 |
erdOne author:erdOne |
chore(RingTheory): add `@[ext]` to `Ideal.Quotient.algHom_ext` |
See [`Ideal.Quotient.ringHom_ext`](https://leanprover-community.github.io/mathlib4_docs/find/?pattern=Ideal.Quotient.ringHom_ext#doc) which also has @[ext 1100].
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
easy
awaiting-author
|
3/2 |
Mathlib/RingTheory/Extension/Presentation/Core.lean,Mathlib/RingTheory/Ideal/Quotient/Operations.lean |
2 |
6 |
['erdOne', 'github-actions', 'j-loreaux'] |
nobody |
28-50909 28 days ago |
28-50909 28 days ago |
3-12761 3 days |
| 31340 |
kim-em author:kim-em |
feat: helper script to summarize CI errors |
---
[](https://gitpod.io/from-referrer/)
|
CI |
235/0 |
scripts/README.md,scripts/failing_ci.py |
2 |
1 |
['github-actions'] |
nobody |
28-26768 28 days ago |
28-26770 28 days ago |
0-0 0 seconds |
| 31348 |
PatrickMassot author:PatrickMassot |
chore: fix a docstring typo |
---
[](https://gitpod.io/from-referrer/)
|
t-analysis
easy
awaiting-author
documentation
|
1/1 |
Mathlib/Analysis/Calculus/Darboux.lean |
1 |
3 |
['ADedecker', 'dopamine333', 'github-actions'] |
nobody |
27-66123 27 days ago |
27-66123 27 days ago |
0-21655 6 hours |
| 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 |
24-66932 24 days ago |
165-81867 5 months ago |
1-60053 1 day |
| 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/)
|
awaiting-CI
t-meta
|
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 |
23-78400 23 days ago |
23-78401 23 days ago |
72-68717 72 days |
| 29257 |
harahu author:harahu |
doc: attach "pre", "pseudo", "semi" and "sub" as a prefixes where they are now free-standing |
These are all examples of [bound morphemes](https://en.wikipedia.org/wiki/Bound_and_free_morphemes) and should be attached, either in closed form or by hyphen, to some other construct.
Whether to write the resulting words in closed form or with a hyphen is a stylistic choice and I am open to discussing the specifics, should that be of interest. I've made choices based on existing literature and what I personally found natural, but other opinions are welcome.
---
[](https://gitpod.io/from-referrer/)
|
t-meta |
42/42 |
Mathlib/Algebra/Star/NonUnitalSubsemiring.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 |
15 |
6 |
['euprunin', 'github-actions', 'harahu', 'mathlib4-merge-conflict-bot'] |
JovanGerb assignee:JovanGerb |
23-33981 23 days ago |
25-50788 25 days ago |
0-0 0 seconds |
| 29458 |
LiamSchilling author:LiamSchilling |
feat(MvPolynomial/WeightedHomogenous): relate `weightedTotalDegree` to `degrees` and `degreeOf` |
`weightedTotalDegree` is the most general notion of multivariate degree in mathlib. These theorems show that it specializes to `degrees` and `degreeOf` with specialized weights.
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
new-contributor
awaiting-author
|
17/0 |
Mathlib/RingTheory/MvPolynomial/Homogeneous.lean |
1 |
6 |
['LiamSchilling', 'chrisflav', 'github-actions'] |
chrisflav assignee:chrisflav |
22-22134 22 days ago |
72-79075 2 months ago |
14-19311 14 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 |
5 |
['faenuccio', 'github-actions', 'grunweg', 'yhx-12243'] |
nobody |
21-83585 21 days ago |
106-67757 3 months ago |
0-1 1 second |
| 30039 |
JovanGerb author:JovanGerb |
feat(push): `push` annotations for `Real.log` |
This PR adds `push` annotations, and tests for `Real.log`.
It also updates the `#push` and `#pull` commands so that they can take a discharger, and can take any head.
---
[](https://gitpod.io/from-referrer/)
|
t-meta
awaiting-author
|
47/18 |
Mathlib/Analysis/SpecialFunctions/Log/Basic.lean,Mathlib/Analysis/SpecialFunctions/Pow/Real.lean,Mathlib/Tactic/Push.lean,MathlibTest/push.lean |
4 |
9 |
['JovanGerb', 'github-actions', 'grunweg', 'mathlib4-merge-conflict-bot'] |
grunweg assignee:grunweg |
21-65107 21 days ago |
23-66397 23 days ago |
28-41247 28 days |
| 31601 |
BoltonBailey author:BoltonBailey |
feat(Data/Nat/Choose): A new strictly positive binomial coefficient |
This is an experimental PR relating to replacing `Nat.choose` with a strictly positive function equivalently to `Nat.choose a (a + b)`
---
[](https://gitpod.io/from-referrer/)
|
t-data |
66/0 |
Mathlib/Data/Nat/Choose/Binomial.lean |
1 |
1 |
['github-actions'] |
nobody |
21-44974 21 days ago |
21-45012 21 days 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.
edit: This lemma should be written using iff (or =), so that we can use it specifically when rewriting with a symmetric relation. Supporting equality in `gcongr` is still work in progress.
---
[](https://gitpod.io/from-referrer/)
|
t-data
delegated
|
5/0 |
Mathlib/Data/Int/ModEq.lean |
1 |
3 |
['fpvandoorn', 'github-actions', 'mathlib-bors'] |
nobody |
20-77343 20 days ago |
174-63623 5 months ago |
1-19951 1 day |
| 31582 |
ADedecker author:ADedecker |
chore: more flavours of derivatives within the empty set |
---
[](https://gitpod.io/from-referrer/)
|
t-analysis
awaiting-CI
|
33/11 |
Mathlib/Analysis/Analytic/Basic.lean,Mathlib/Analysis/Analytic/Constructions.lean,Mathlib/Analysis/Analytic/ConvergenceRadius.lean,Mathlib/Analysis/Analytic/Within.lean,Mathlib/Analysis/Calculus/FDeriv/Basic.lean,Mathlib/Analysis/Calculus/FDeriv/Const.lean |
6 |
4 |
['github-actions', 'grunweg'] |
grunweg assignee:grunweg |
20-57746 20 days ago |
20-57746 20 days ago |
0-0 0 seconds |
| 31607 |
grunweg author:grunweg |
chore: rename `continuous{,On,At,Within}_const to `ContinuousFoo.const` |
Needs fixing all remaining deprecation warnings.
Zulip discussion: [#mathlib4 > Naming convention @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Naming.20convention/near/447491526)
---
[](https://gitpod.io/from-referrer/)
|
awaiting-CI
delegated
|
86/82 |
Archive/Hairer.lean,Mathlib/Analysis/BoxIntegral/Box/Basic.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Unital.lean,Mathlib/Analysis/Calculus/Deriv/MeanValue.lean,Mathlib/Analysis/Calculus/DiffContOnCl.lean,Mathlib/Analysis/Calculus/MeanValue.lean,Mathlib/Analysis/Calculus/Taylor.lean,Mathlib/Analysis/Complex/AbsMax.lean,Mathlib/Analysis/Complex/CauchyIntegral.lean,Mathlib/Analysis/Complex/PhragmenLindelof.lean,Mathlib/Analysis/Complex/RemovableSingularity.lean,Mathlib/Analysis/Convex/Exposed.lean,Mathlib/Analysis/Convex/Gauge.lean,Mathlib/Analysis/Convex/PartitionOfUnity.lean,Mathlib/Analysis/Convolution.lean,Mathlib/Analysis/Normed/Module/Ball/Homeomorph.lean,Mathlib/Analysis/Normed/Operator/BoundedLinearMaps.lean,Mathlib/Analysis/ODE/PicardLindelof.lean,Mathlib/Analysis/SpecialFunctions/Gamma/Basic.lean,Mathlib/Analysis/SpecialFunctions/Integrability/Basic.lean,Mathlib/Analysis/SpecialFunctions/Pow/Continuity.lean,Mathlib/MeasureTheory/Integral/Bochner/Basic.lean,Mathlib/MeasureTheory/Integral/CircleIntegral.lean,Mathlib/MeasureTheory/Integral/CircleTransform.lean,Mathlib/MeasureTheory/Integral/IntervalIntegral/Basic.lean,Mathlib/MeasureTheory/Integral/IntervalIntegral/FundThmCalculus.lean,Mathlib/MeasureTheory/Integral/RieszMarkovKakutani/Real.lean,Mathlib/NumberTheory/LSeries/PrimesInAP.lean,Mathlib/NumberTheory/NumberField/CanonicalEmbedding/NormLeOne.lean,Mathlib/Topology/Algebra/ContinuousMonoidHom.lean,Mathlib/Topology/Algebra/GroupWithZero.lean,Mathlib/Topology/Algebra/Indicator.lean,Mathlib/Topology/Algebra/Order/Floor.lean,Mathlib/Topology/Connected/Basic.lean,Mathlib/Topology/Constructions.lean,Mathlib/Topology/Constructions/SumProd.lean,Mathlib/Topology/Continuous.lean,Mathlib/Topology/ContinuousOn.lean,Mathlib/Topology/FiberBundle/Basic.lean,Mathlib/Topology/Hom/ContinuousEval.lean,Mathlib/Topology/Homeomorph/Defs.lean,Mathlib/Topology/Order.lean,Mathlib/Topology/Order/IntermediateValue.lean,Mathlib/Topology/VectorBundle/Basic.lean |
44 |
3 |
['github-actions', 'j-loreaux', 'mathlib-bors'] |
nobody |
20-1847 20 days ago |
20-12869 20 days ago |
0-1 1 second |
| 30526 |
SnirBroshi author:SnirBroshi |
chore(Logic/Relation): use `Subrelation` to state theorems |
chore(Logic/Relation): replace every `∀ x y, r x y → r' x y` with `Subrelation r r'`
---
[](https://gitpod.io/from-referrer/)
|
awaiting-zulip |
79/73 |
Mathlib/CategoryTheory/IsConnected.lean,Mathlib/CategoryTheory/Limits/Types/Coequalizers.lean,Mathlib/CategoryTheory/Limits/Types/Filtered.lean,Mathlib/Data/Setoid/Basic.lean,Mathlib/GroupTheory/FreeGroup/Basic.lean,Mathlib/Logic/Relation.lean,Mathlib/Order/Interval/Finset/Basic.lean |
7 |
5 |
['SnirBroshi', 'github-actions', 'mathlib4-merge-conflict-bot', 'thorimur', 'vihdzp'] |
thorimur assignee:thorimur |
17-60586 17 days ago |
17-60606 17 days ago |
8-76821 8 days |
| 31637 |
Whysoserioushah author:Whysoserioushah |
feat(Data/Matrix/Basis): add some lemmas |
Zulip discussion : https://leanprover.zulipchat.com/#narrow/channel/217875-Is-there-code-for-X.3F/topic/Matrix.2Eone_eq_sum_single.3F/with/555689472
---
[](https://gitpod.io/from-referrer/)
|
t-data
awaiting-author
|
14/0 |
Mathlib/Data/Matrix/Basis.lean |
1 |
9 |
['Whysoserioushah', 'eric-wieser', 'github-actions', 'kckennylau'] |
nobody |
17-60409 17 days ago |
17-60409 17 days ago |
2-60442 2 days |
| 30562 |
dwrensha author:dwrensha |
fix(Data/Fintype/Perm): make the main logic of Equiv.instFintype irreducible |
Adds a new `irreducible_def` for the main branch of `Equiv.instFintype` to avoid errors about deep recursion.
This is an update of #15045 and #30560 according to the discussion in those PRs and in [this zulip thread](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/kernel.20deep.20recursion.20detected/near/454301820).
---
[](https://gitpod.io/from-referrer/)
|
t-data
awaiting-author
|
40/8 |
Mathlib/Combinatorics/Derangements/Finite.lean,Mathlib/Data/Fintype/Perm.lean,Mathlib/LinearAlgebra/Matrix/SpecialLinearGroup.lean,MathlibTest/MatrixDetOne.lean |
4 |
16 |
['dwrensha', 'github-actions', 'leanprover-bot', 'plp127', 'robin-carlier'] |
robin-carlier assignee:robin-carlier |
17-56478 17 days ago |
38-64757 1 month ago |
12-56370 12 days |
| 26885 |
pechersky author:pechersky |
feat(Topology/ValuativeRel): ValuativeTopology 𝒪[K] |
and even when not a field, `ValuativeRel 𝒪[K]`
This is an example of something achievable with the new declarations that wasn't possible with Valued
Such that we can discuss the valuations on the subring without always using coercions
But to achieve this, one needs some juggling of the value groups
---
[](https://gitpod.io/from-referrer/)
- [x] depends on: #26834
- [ ] depends on : #30135
|
t-algebra
t-topology
t-number-theory
label:t-algebra$ |
66/0 |
Mathlib/Topology/Algebra/Valued/ValuativeRel.lean |
1 |
10 |
['erdOne', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'pechersky'] |
alreadydone assignee:alreadydone |
17-50338 17 days ago |
17-50361 17 days ago |
149-18389 149 days |
| 31326 |
sgouezel author:sgouezel |
chore: deprecate `smooth` variants of `contMDiff` results |
---
[](https://gitpod.io/from-referrer/)
|
t-differential-geometry
awaiting-author
|
44/52 |
Mathlib/Analysis/Calculus/BumpFunction/FiniteDimension.lean,Mathlib/Geometry/Manifold/PartitionOfUnity.lean |
2 |
6 |
['github-actions', 'grunweg', 'sgouezel'] |
grunweg assignee:grunweg |
17-39845 17 days ago |
17-55764 17 days ago |
8-84793 8 days |
| 31386 |
harahu author:harahu |
doc: demote repeated H1 headers to H2 |
---
[](https://gitpod.io/from-referrer/)
|
|
216/0 |
scripts/demote_docstring_headers.py,scripts/find_docstring_headers.py |
2 |
6 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
17-33411 17 days ago |
17-33435 17 days ago |
0-0 0 seconds |
| 12032 |
mcdoll author:mcdoll |
feat: delta distribution as a limit |
---
- [ ] depends on: #11496
[](https://gitpod.io/from-referrer/)
|
t-analysis
WIP
|
58/0 |
Mathlib/Analysis/Distribution/DiracDelta.lean |
1 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
17-18183 17 days ago |
unknown |
unknown |
| 24965 |
erdOne author:erdOne |
refactor: Make `IsLocalHom` take unbundled map |
Under the current definition, `IsLocalHom f` and `IsLocalHom f.toMonoidHom` are not defeq, which causes quite some annoyances. We also have a consensus to not use `*HomClass` in definitions. As a result, we change `IsLocalHom` to take an unbundled function instead of a funlike.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
delegated
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 |
12 |
['adomani', 'alreadydone', 'erdOne', 'eric-wieser', 'github-actions', 'jcommelin', 'leanprover-community-bot-assistant', 'mathlib-bors'] |
mattrobball assignee:mattrobball |
16-83310 16 days ago |
16-83310 16 days ago |
24-84527 24 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'] |
nobody |
16-52023 16 days ago |
129-31203 4 months ago |
146-23504 146 days |
| 30842 |
kim-em author:kim-em |
feat: add Aristotle task for command palette |
---
[](https://gitpod.io/from-referrer/)
|
CI |
128/0 |
.vscode/tasks.json,scripts/README.md,scripts/aristotle/README.md |
3 |
17 |
['eric-wieser', 'euprunin', 'github-actions', 'kim-em', 'vikram-shanker'] |
bryangingechen assignee:bryangingechen |
16-26030 16 days ago |
42-15378 1 month ago |
42-15417 42 days |
| 30988 |
erdOne author:erdOne |
feat(AlgebraicGeometry): descending affine cover of an inverse limit |
---
[](https://gitpod.io/from-referrer/)
|
t-algebraic-geometry |
347/35 |
Mathlib/Algebra/Category/Ring/Constructions.lean,Mathlib/AlgebraicGeometry/AffineTransitionLimit.lean,Mathlib/AlgebraicGeometry/Gluing.lean,Mathlib/AlgebraicGeometry/Morphisms/IsIso.lean,Mathlib/AlgebraicGeometry/Pullbacks.lean,Mathlib/AlgebraicGeometry/QuasiAffine.lean,Mathlib/AlgebraicGeometry/Sites/MorphismProperty.lean,Mathlib/Topology/LocalAtTarget.lean |
8 |
22 |
['chrisflav', 'erdOne', 'github-actions', 'mathlib4-merge-conflict-bot'] |
alexjbest assignee:alexjbest |
15-84877 15 days ago |
15-84885 15 days ago |
38-143 38 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/)
|
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 |
11 |
['Ruben-VandeVelde', 'YaelDillies', 'github-actions', 'mathlib4-merge-conflict-bot'] |
bryangingechen assignee:bryangingechen |
15-78104 15 days ago |
15-78112 15 days ago |
2-29376 2 days |
| 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
|
211/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 |
22 |
['YaelDillies', 'github-actions', 'kbuzzard', 'leanprover-community-bot-assistant', 'mathlib4-merge-conflict-bot', 'sgouezel'] |
nobody |
15-76774 15 days ago |
15-76790 15 days ago |
8-77637 8 days |
| 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
|
220/6 |
Mathlib.lean,Mathlib/MeasureTheory/Function/LpSeminorm/Defs.lean,Mathlib/MeasureTheory/Function/LpSeminorm/NNLpNorm.lean,Mathlib/MeasureTheory/Function/LpSeminorm/TriangleInequality.lean |
4 |
21 |
['YaelDillies', 'b-mehta', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-merge-conflict-bot', 'sgouezel'] |
nobody |
15-76566 15 days ago |
15-76580 15 days ago |
13-15316 13 days |
| 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
|
75/0 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Simproc/DivisorsAntidiag.lean |
3 |
9 |
['YaelDillies', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
15-75435 15 days ago |
15-75451 15 days ago |
0-260 4 minutes |
| 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
|
21/3 |
Mathlib/Topology/Algebra/ConstMulAction.lean,Mathlib/Topology/Algebra/Group/Quotient.lean |
2 |
5 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
15-75379 15 days ago |
35-46981 1 month ago |
0-352 5 minutes |
| 15443 |
YaelDillies author:YaelDillies |
feat: 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 |
40 |
['Parcly-Taxel', 'YaelDillies', 'b-mehta', 'github-actions', 'hrmacbeth', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'sgouezel'] |
nobody |
15-75091 15 days ago |
15-75108 15 days ago |
89-28229 89 days |
| 31263 |
LiranShaul author:LiranShaul |
feat: arbitrary product of injective modules is injective |
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-algebra
awaiting-author
label:t-algebra$ |
15/0 |
Mathlib/Algebra/Module/Injective.lean |
1 |
12 |
['LiranShaul', 'erdOne', 'github-actions', 'joelriou', 'kbuzzard', 'mathlib4-merge-conflict-bot'] |
nobody |
15-70319 15 days ago |
15-77207 15 days ago |
0-21724 6 hours |
| 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`.
---
- [x] depends on: #30287
[](https://gitpod.io/from-referrer/)
|
t-combinatorics
awaiting-author
|
93/0 |
Mathlib/Combinatorics/SimpleGraph/Bipartite.lean |
1 |
23 |
['YaelDillies', 'b-mehta', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'mitchell-horner', 'vlad902'] |
YaelDillies assignee:YaelDillies |
15-68977 15 days ago |
15-72689 15 days ago |
78-11533 78 days |
| 31590 |
SuccessMoses author:SuccessMoses |
chore: tag `commutatorElement_def` with `simp` |
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-algebra
awaiting-author
label:t-algebra$ |
1/0 |
Mathlib/Algebra/Group/Commutator.lean |
1 |
2 |
['github-actions', 'grunweg'] |
nobody |
15-61377 15 days ago |
15-61377 15 days ago |
6-8213 6 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 |
53 |
['b-mehta', 'espottesmith', 'github-actions', 'jt496', 'lauramonk', 'mathlib4-merge-conflict-bot'] |
b-mehta assignee:b-mehta |
15-61289 15 days ago |
15-61311 15 days ago |
96-38544 96 days |
| 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
|
145/0 |
Mathlib/AlgebraicTopology/Anodyne.lean,Mathlib/AlgebraicTopology/KanFibration.lean,Mathlib/CategoryTheory/MorphismProperty/WeakSaturation.lean |
3 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
15-61284 15 days ago |
15-61303 15 days ago |
0-2 2 seconds |
| 29744 |
espottesmith author:espottesmith |
feat(Combinatorics): define directed hypergraphs |
This PR defines directed hypergraphs:
```
@[ext]
structure DiHypergraph (α : Type*) where
/-- The vertex set -/
vertexSet : Set α
/-- The edge set -/
edgeSet : Set ((Set α) × (Set α))
/-- Each edge is a pair (s, d), where s ⊆ vertexSet and d ⊆ vertexSet -/
edge_src_dst_isSubset_vertexSet' : ∀ ⦃e⦄, e ∈ edgeSet → e.1 ⊆ vertexSet ∧ e.2 ⊆ vertexSet
```
Additional definitions:
- tail/head stars and negative/positive stars
- some special cases (B-Graph, F-Graph, BF-Graph, and what I'm calling a "non-endless" dihypergraph, where neither the source/tail nor the destination/head are empty)
- Vertex and (hyper)edge adjacency
- isolated vertices
- empty and nonempty dihypergraphs
The design employed here is based off of #28613, but this PR does not depend on that one.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-combinatorics
|
391/0 |
Mathlib.lean,Mathlib/Combinatorics/DiHypergraph/Basic.lean |
2 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
b-mehta assignee:b-mehta |
15-61243 15 days ago |
15-61269 15 days ago |
78-49667 78 days |
| 6859 |
MohanadAhmed author:MohanadAhmed |
feat: 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 |
15-60620 15 days ago |
828-29333 2 years 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 |
15-60453 15 days ago |
513-67166 1 year 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 |
15-60351 15 days ago |
282-71311 9 months ago |
87-64575 87 days |
| 23772 |
SEU-Prime author:SEU-Prime |
feat: Amice equivalence |
i built amice equiv
[](https://gitpod.io/from-referrer/)
|
t-number-theory
WIP
|
283/0 |
Mathlib/NumberTheory/Padics/Amice.lean |
1 |
2 |
['grunweg'] |
nobody |
15-60244 15 days ago |
241-65290 7 months ago |
0-8688 2 hours |
| 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 |
15-60154 15 days ago |
99-1542 3 months ago |
118-2181 118 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 |
15-60131 15 days ago |
179-4155 5 months ago |
20-11468 20 days |
| 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 |
15-60121 15 days ago |
179-4180 5 months ago |
20-7584 20 days |
| 26013 |
tsuki8 author:tsuki8 |
feat(Data/Finset/Card,Data/Set/Finite/Basic): TODO needs a better title |
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 |
15-60069 15 days ago |
156-83292 5 months ago |
13-85893 13 days |
| 26881 |
emo916math author:emo916math |
feat(Analysis/Calculus/Deriv/Star): a formula for `deriv (conj ∘ f ∘ conj)` |
Added a lemma that `deriv (conj ∘ f ∘ conj) = conj ∘ deriv f ∘ conj`, proved by cases on whether the derivative mathematically exists or not. This PR replaces [#26805](https://github.com/leanprover-community/mathlib4/pull/26805); see discussion there.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-analysis
awaiting-author
|
50/2 |
Mathlib/Analysis/Calculus/Deriv/Star.lean |
1 |
15 |
['emo916math', 'github-actions', 'j-loreaux', 'kckennylau'] |
j-loreaux assignee:j-loreaux |
15-59924 15 days ago |
118-59672 3 months ago |
31-70593 31 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
awaiting-author
|
22/0 |
Mathlib/Data/Rat/Lemmas.lean |
1 |
33 |
['github-actions', 'kim-em', 'mathlib-bors', 'pechersky', 'sinianluoye', 'themathqueen'] |
pechersky assignee:pechersky |
15-59841 15 days ago |
39-18903 1 month ago |
80-3629 80 days |
| 29921 |
mans0954 author:mans0954 |
refactor(RingTheory/Polynomial/SmallDegreeVieta): convert to {p : R[X]} (hp : p.natDegree = 2) |
Convert `RingTheory/Polynomial/SmallDegreeVieta` from `{a b c : R} (C a * X ^ 2 + C b * X + C c)` to `{p : R[X]} (hp : p.natDegree = 2)`
(see [Zulip discussion](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/discriminants.20of.20low.20degree.20polynomials/with/538010519))
---
- [x] depends on: #29981
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
awaiting-author
|
75/60 |
Mathlib/RingTheory/Polynomial/SmallDegreeVieta.lean |
1 |
14 |
['JovanGerb', 'chrisflav', 'github-actions', 'kckennylau', 'mans0954', 'mathlib4-dependent-issues-bot', 'vihdzp'] |
erdOne assignee:erdOne |
15-59667 15 days ago |
40-76900 1 month ago |
17-62236 17 days |
| 29361 |
FlAmmmmING author:FlAmmmmING |
feat: Catalan generating function as a formal power series |
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
awaiting-author
|
56/0 |
Mathlib.lean,Mathlib/RingTheory/PowerSeries/Catalan.lean |
2 |
10 |
['FlAmmmmING', 'Ruben-VandeVelde', 'github-actions', 'kbuzzard', 'mathlib4-merge-conflict-bot', 'wwylele'] |
kbuzzard assignee:kbuzzard |
15-48684 15 days ago |
15-67300 15 days ago |
70-34394 70 days |
| 30609 |
FlAmmmmING author:FlAmmmmING |
feat(Combinatorics/Enumerative/Catalan): large and small Schröder numbers |
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-combinatorics
awaiting-author
|
128/1 |
Mathlib/Combinatorics/Enumerative/Catalan.lean |
1 |
6 |
['FlAmmmmING', 'SnirBroshi', 'YaelDillies', 'github-actions', 'mathlib4-merge-conflict-bot', 'plp127'] |
nobody |
15-46951 15 days ago |
15-67241 15 days ago |
17-66663 17 days |
| 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
awaiting-author
label:t-algebra$ |
182/0 |
Mathlib/Algebra/CharP/Invertible.lean,Mathlib/RingTheory/RootsOfUnity/Complex.lean |
2 |
3 |
['github-actions', 'mans0954', 'urkud'] |
jcommelin assignee:jcommelin |
15-46510 15 days ago |
15-46510 15 days ago |
157-25048 157 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
awaiting-author
|
13/0 |
Mathlib/MeasureTheory/PiSystem.lean |
1 |
14 |
['EtienneC30', 'KiringYJ', 'dagurtomas', 'github-actions', 'ocfnash'] |
RemyDegenne assignee:RemyDegenne |
15-46017 15 days ago |
15-46017 15 days ago |
138-3922 138 days |
| 31719 |
maksym-radziwill author:maksym-radziwill |
feat: Borel-Caratheodory (2nd revision) |
This proves the Borel-Caratheodory theorem, for the previous iteration see https://github.com/leanprover-community/mathlib4/pull/30424
CC: @grunweg @j-loreaux @Ruben-VandeVelde @wwylele
---
[](https://gitpod.io/from-referrer/)
|
t-analysis
awaiting-author
|
146/0 |
Mathlib.lean,Mathlib/Analysis/Complex/BorelCaratheodory.lean,docs/1000.yaml |
3 |
4 |
['github-actions', 'grunweg', 'maksym-radziwill', 'mathlib4-merge-conflict-bot'] |
nobody |
15-26779 15 days ago |
15-26803 15 days ago |
0-35115 9 hours |
| 30953 |
kim-em author:kim-em |
experiment: add `canonical` to Mathlib |
Depends on (these must be merged first before CI will succeed here)
- [x] #30952
- [x] #30844 |
|
63/3 |
Mathlib/Tactic/Common.lean,Mathlib/Tactic/Linter/DirectoryDependency.lean,MathlibTest/canonical.lean,lake-manifest.json,lakefile.lean |
5 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
15-18567 15 days ago |
15-18581 15 days ago |
0-0 0 seconds |
| 30190 |
joelriou author:joelriou |
feat(CategoryTheory/Sites): functoriality of descent data |
Given a pseudofunctor `F` from `LocallyDiscrete Cᵒᵖ` to `Cat`, we show that up to an equivalence, the category `F.DescentData f` is unchanged when we replace `S` by an isomorphic object, or the family `f i : X i ⟶ S` by another family which generates the same sieve (see `Pseudofunctor.pullFunctorEquivalence`).
Co-authored-by: Christian Merten [christian@merten.dev](mailto:christian@merten.dev)
---
- [x] depends on: #25971
- [x] depends on: #30177
- [x] depends on: #30189
[](https://gitpod.io/from-referrer/)
|
t-category-theory
WIP
|
243/1 |
Mathlib/CategoryTheory/Bicategory/Functor/Cat.lean,Mathlib/CategoryTheory/Sites/Descent/DescentData.lean |
2 |
5 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
14-71921 14 days ago |
14-72008 14 days ago |
0-2 2 seconds |
| 29409 |
Julian author:Julian |
feat(Mathlib/Analysis): deriv_eq_self and deriv_exp_iff |
---
[](https://gitpod.io/from-referrer/)
|
t-analysis
awaiting-author
|
29/0 |
Mathlib/Analysis/SpecialFunctions/ExpDeriv.lean |
1 |
9 |
['Julian', 'Paul-Lez', 'eric-wieser', 'github-actions', 'j-loreaux', 'mathlib4-merge-conflict-bot'] |
j-loreaux assignee:j-loreaux |
14-59982 14 days ago |
14-59998 14 days ago |
15-76317 15 days |
| 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
|
119/4 |
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 |
18 |
['adomani', 'b-mehta', 'eric-wieser', 'github-actions', 'grunweg', 'kim-em', 'mathlib-bors', 'mathlib4-merge-conflict-bot'] |
nobody |
14-41141 14 days ago |
14-41158 14 days ago |
15-14325 15 days |
| 31611 |
thorimur author:thorimur |
feat(Meta): `withPlural` wrapper for more readable messages in source |
This small PR introduces a thin wrapper `withPlural` for Lean's textual datatypes so that we can write
```
"foo".withPlural "foos" count
```
instead of
```
if count = 1 then "foo" else "foos"
```
The dot notation here is chosen so that the singular version of the word appears at the start of the syntax, as opposed to buried in an `if/then`. This makes dynamically pluralizing a word in `MessageData` (which is a relatively common occurrence) a bit easier to read in source, especially when multiple pluralizations are needed close to one another.
---
Am I handling the copyright header correctly? My reasoning is that the file was devoid of content, and so this is ultimately a new file. But I'm not sure this is technically what should happen here.
[](https://gitpod.io/from-referrer/)
|
maintainer-merge
t-meta
|
63/5 |
Mathlib/Lean/Message.lean |
1 |
17 |
['adomani', 'github-actions', 'grunweg', 'mathlib4-merge-conflict-bot', 'thorimur'] |
alexjbest assignee:alexjbest |
14-30507 14 days ago |
15-25403 15 days ago |
20-52351 20 days |
| 29953 |
slashbade author:slashbade |
feat: add reap for experiment |
---
[](https://gitpod.io/from-referrer/)
|
new-contributor |
40/3 |
Cache/IO.lean,Mathlib/Tactic/Common.lean,Mathlib/Tactic/Linter/DirectoryDependency.lean,lake-manifest.json,lakefile.lean |
5 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
14-11227 14 days ago |
14-72017 14 days ago |
0-0 0 seconds |
| 31854 |
erdOne author:erdOne |
chore(AlgebraicGeometry): API for `𝒪ₓ`-modules |
---
[](https://gitpod.io/from-referrer/)
|
t-algebraic-geometry
awaiting-author
|
475/15 |
Mathlib/Algebra/Category/ModuleCat/ChangeOfRings.lean,Mathlib/Algebra/Category/ModuleCat/Presheaf/Colimits.lean,Mathlib/Algebra/Category/ModuleCat/Presheaf/Limits.lean,Mathlib/Algebra/Category/ModuleCat/Sheaf/Colimits.lean,Mathlib/Algebra/Category/ModuleCat/Sheaf/PullbackContinuous.lean,Mathlib/Algebra/Category/ModuleCat/Sheaf/PushforwardContinuous.lean,Mathlib/AlgebraicGeometry/Modules/Sheaf.lean,Mathlib/AlgebraicGeometry/OpenImmersion.lean |
8 |
3 |
['erdOne', 'github-actions', 'joelriou'] |
nobody |
13-78753 13 days ago |
13-78753 13 days ago |
0-69692 19 hours |
| 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 |
789/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 |
33 |
['FLDutchmann', 'JovanGerb', 'github-actions', 'grunweg', 'mathlib4-merge-conflict-bot', 'xyzw12345'] |
JovanGerb assignee:JovanGerb |
13-75694 13 days ago |
13-75712 13 days ago |
132-58204 132 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
awaiting-author
|
124/0 |
Mathlib/Analysis/Normed/Group/Basic.lean,Mathlib/Topology/MetricSpace/Basic.lean,Mathlib/Topology/MetricSpace/Pseudo/Constructions.lean |
3 |
12 |
['github-actions', 'kckennylau', 'mathlib4-merge-conflict-bot', 'pechersky'] |
urkud assignee:urkud |
13-61242 13 days ago |
13-61242 13 days ago |
114-37138 114 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 |
8/8 |
Mathlib/Data/Finset/Max.lean |
1 |
7 |
['eric-wieser', 'github-actions', 'jcommelin', 'kckennylau', 'mathlib-bors'] |
pechersky assignee:pechersky |
13-58869 13 days ago |
13-58876 13 days ago |
88-23711 88 days |
| 31597 |
grunweg author:grunweg |
chore(AtLocation): allow throwing a warning when no progress is being made |
A future PR will use this to make `by_contra!` and friends warn if the `push_neg` step makes no progress.
Co-authored by: Jovan Gerbscheid
---
[](https://gitpod.io/from-referrer/)
|
t-meta
awaiting-author
|
46/28 |
Mathlib/Tactic/Abel.lean,Mathlib/Tactic/Field.lean,Mathlib/Tactic/FieldSimp.lean,Mathlib/Tactic/NormNum/Core.lean,Mathlib/Tactic/Push.lean,Mathlib/Tactic/ReduceModChar.lean,Mathlib/Tactic/Ring/RingNF.lean,Mathlib/Util/AtLocation.lean,MathlibTest/FieldSimp.lean,MathlibTest/abel.lean |
10 |
6 |
['JovanGerb', 'fpvandoorn', 'github-actions', 'thorimur'] |
thorimur assignee:thorimur |
13-55339 13 days ago |
13-55339 13 days ago |
7-68323 7 days |
| 30678 |
YaelDillies author:YaelDillies |
refactor(Algebra/Quaternion): intermediate `Module` instance |
This `Module` instance allows me to not ungeneralise the `NoZeroSMulDivisors R ℍ[R,c₁,c₂,c₃]` in #30563.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
45/28 |
Mathlib/Algebra/Quaternion.lean |
1 |
24 |
['YaelDillies', 'eric-wieser', 'github-actions', 'kckennylau', 'leanprover-bot', 'leanprover-radar'] |
joneugster assignee:joneugster |
13-54295 13 days ago |
45-83367 1 month ago |
46-21706 46 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 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
13-44327 13 days ago |
13-63700 13 days ago |
85-57202 85 days |
| 30436 |
wwylele author:wwylele |
feat(Topology/InfiniteSum): tprod_one_{add/sub}_ordered |
This extends the existing `Finset.prod_one_sub_ordered` to infinite sum/product, and also adds the more natural `add` version.
Together with some previous PRs about infinite sum/prod and powerseries, this is part of my effort of upstreaming useful stuff from https://github.com/wwylele/PentagonalNumberTheorem. It starts getting into niche lemma, so suggestions such that not wanting this in mathlib, or it should be stated in a different form, are all welcomed.
---
[](https://gitpod.io/from-referrer/)
|
t-topology
awaiting-author
|
44/0 |
Mathlib/Algebra/BigOperators/Ring/Finset.lean,Mathlib/Topology/Algebra/InfiniteSum/Ring.lean |
2 |
5 |
['github-actions', 'kckennylau', 'wwylele'] |
grunweg assignee:grunweg |
13-37558 13 days ago |
13-39777 13 days ago |
41-31045 41 days |
| 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: #xyz [optional extra text]
-->
[](https://gitpod.io/from-referrer/)
|
new-contributor
awaiting-author
|
70/1 |
Mathlib/Analysis/LocallyConvex/Separation.lean,Mathlib/Analysis/RCLike/Lemmas.lean,Mathlib/Topology/Order/OrderClosed.lean |
3 |
16 |
['faenuccio', 'fpvandoorn', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'mcdoll', 'themathqueen', 'yuanyi-350'] |
faenuccio assignee:faenuccio |
13-16394 13 days ago |
13-23838 13 days ago |
21-29486 21 days |
| 29856 |
mans0954 author:mans0954 |
feat(Analysis/Normed/Ring/Basic): Add NonUnitalNonAssocSeminormedRing and NonUnitalNonAssocNormedRing |
Adds the classes `NonUnitalNonAssocSeminormedRing` and `NonUnitalNonAssocNormedRing` and relaxes the `NonUnitalSeminormedRing` section to `NonUnitalNonAssocSeminormedRing`.
Examples of non-unital non-associative normed rings include non-untial JB-algebras and non-unital JB*-algebras.
---
[](https://gitpod.io/from-referrer/)
|
t-analysis
awaiting-author
|
110/11 |
Mathlib/Analysis/Normed/Ring/Basic.lean,MathlibTest/TCSynth.lean |
2 |
15 |
['github-actions', 'j-loreaux', 'leanprover-bot'] |
ADedecker assignee:ADedecker |
13-16158 13 days ago |
16-36702 16 days ago |
58-29334 58 days |
| 27254 |
yuanyi-350 author:yuanyi-350 |
feat: 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 |
29 |
['github-actions', 'jsm28', 'kbuzzard', 'leanprover-community-bot-assistant', 'madvorak', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'themathqueen', 'wwylele', 'yuanyi-350'] |
jsm28 assignee:jsm28 |
12-81973 12 days ago |
12-81992 12 days ago |
123-83644 123 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
awaiting-zulip
|
5/11 |
Mathlib/RingTheory/Bialgebra/Hom.lean |
1 |
16 |
['YaelDillies', 'erdOne', 'eric-wieser', 'github-actions'] |
alreadydone assignee:alreadydone |
12-70329 12 days ago |
12-70329 12 days ago |
101-9047 101 days |
| 30637 |
strihanje01 author:strihanje01 |
feat(Combinatorics/SetFamily/Lindstrom): Lindstrom's theorem for subfamilies with equal unions |
add Lindstrom's theorem and its strengthening for equal intersections
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-combinatorics
|
209/0 |
Mathlib/Combinatorics/SetFamily/Lindstrom.lean |
1 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
b-mehta assignee:b-mehta |
12-68166 12 days ago |
13-50597 13 days ago |
46-17607 46 days |
| 31259 |
YaelDillies author:YaelDillies |
refactor(Dynamics): use `SetRel` notions of separation and cover |
... instead of the handmade ones.
---
[](https://gitpod.io/from-referrer/)
|
t-dynamics |
173/203 |
Mathlib/Data/Rel/Cover.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/Topology/UniformSpace/Defs.lean |
7 |
7 |
['D-Thomine', 'YaelDillies', 'github-actions', 'mathlib4-merge-conflict-bot'] |
urkud assignee:urkud |
12-60894 12 days ago |
15-72465 15 days ago |
28-74394 28 days |
| 31949 |
ADedecker author:ADedecker |
chore: prefer `Pi.single i 1 j` over `fun j => if i = j then 1 else 0` |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
awaiting-author
label:t-algebra$ |
23/21 |
Mathlib/Algebra/BigOperators/Pi.lean,Mathlib/Analysis/Convex/StdSimplex.lean,Mathlib/LinearAlgebra/Matrix/Adjugate.lean,Mathlib/LinearAlgebra/Pi.lean,Mathlib/Topology/Algebra/Module/Basic.lean |
5 |
5 |
['eric-wieser', 'github-actions', 'themathqueen'] |
nobody |
12-34515 12 days ago |
12-34515 12 days ago |
0-21800 6 hours |
| 31965 |
bwangpj author:bwangpj |
feat: fiber of RingHom.specComap |
This contribution was created as part of the Heidelberg Lean workshop "Formalising algebraic geometry" in November 2025.
Co-authored-by: Christian Merten @chrisflav
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
awaiting-author
|
29/0 |
Mathlib/RingTheory/Spectrum/Prime/RingHom.lean |
1 |
3 |
['bwangpj', 'erdOne', 'github-actions'] |
nobody |
12-32792 12 days ago |
12-35518 12 days ago |
0-5921 1 hour |
| 30981 |
jsm28 author:jsm28 |
feat(Geometry/Euclidean/Angle/Bisector): oriented angle bisection mod π |
Add lemmas relating equal distance to two lines to bisecting the angle between them mod π (expressed as usual as equality of twice angles), building on the previous lemmas (#30477) dealing with bisection mod 2π.
---
- [ ] depends on: #30474
- [ ] depends on: #30477
- [ ] depends on: #30600
- [ ] depends on: #30703
[](https://gitpod.io/from-referrer/)
|
t-euclidean-geometry |
146/4 |
Mathlib/Geometry/Euclidean/Angle/Bisector.lean |
1 |
4 |
['github-actions', 'jsm28', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
JovanGerb assignee:JovanGerb |
12-29838 12 days ago |
15-76984 15 days ago |
20-33816 20 days |
| 31525 |
kim-em author:kim-em |
feat: convex combinations in `Set.Icc` |
This will hopefully become obsolete with a more general theory of convex spaces, but this would be helpful to go on for now.
Note: Proofs in this PR were developed with assistance from Claude. |
t-topology
delegated
|
142/0 |
Mathlib/Topology/UnitInterval.lean |
1 |
5 |
['github-actions', 'jcommelin', 'kim-em', 'mathlib-bors'] |
ADedecker assignee:ADedecker |
12-20283 12 days ago |
13-77037 13 days ago |
8-54621 8 days |
| 30877 |
YaelDillies author:YaelDillies |
feat(Algebra/MonoidAlgebra): extend the `R[M]` notation to `MonoidAlgebra R M` |
It currently only is notation for `AddMonoidAlgebra R M`.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
awaiting-author
label:t-algebra$ |
212/161 |
Mathlib/Algebra/MonoidAlgebra/Basic.lean,Mathlib/Algebra/MonoidAlgebra/Defs.lean,Mathlib/Algebra/MonoidAlgebra/Lift.lean,Mathlib/Algebra/MonoidAlgebra/MapDomain.lean,Mathlib/Algebra/MonoidAlgebra/Module.lean,Mathlib/Algebra/MonoidAlgebra/NoZeroDivisors.lean,Mathlib/Algebra/MonoidAlgebra/Opposite.lean,Mathlib/Algebra/MonoidAlgebra/Support.lean,MathlibTest/Algebra/MonoidAlgebra/Defs.lean |
9 |
24 |
['YaelDillies', 'erdOne', 'eric-wieser', 'github-actions', 'mathlib4-merge-conflict-bot', 'vihdzp'] |
kmill assignee:kmill |
12-1977 12 days ago |
12-31168 12 days ago |
25-40830 25 days |
| 31576 |
kim-em author:kim-em |
feat: in a semilocally simply connected, locally path-connected space, the quotient of paths by homotopy has the discrete topology |
This is closely related to, but not quite the same, as the quotient path space with fixed initial point being an even covering (under the endpoint map).
Depends on
- [ ] #31449
- [ ] #31525
- [x] #31574
- [ ] #31575.
Claude wrote most of the text, under my prompting.
|
|
1598/0 |
Mathlib.lean,Mathlib/AlgebraicTopology/FundamentalGroupoid/Basic.lean,Mathlib/AlgebraicTopology/FundamentalGroupoid/SemilocallySimplyConnected.lean,Mathlib/Topology/Connected/PathConnected.lean,Mathlib/Topology/Homotopy/Path.lean,Mathlib/Topology/Path.lean,Mathlib/Topology/UnitInterval.lean |
7 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
11-79444 11 days ago |
15-22567 15 days ago |
0-0 0 seconds |
| 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 de Bruijn-Erdos should move out of this file.
---
[](https://gitpod.io/from-referrer/)
|
t-combinatorics |
131/0 |
Mathlib/Combinatorics/SimpleGraph/DeBruijnErdos.lean |
1 |
1 |
['github-actions'] |
nobody |
11-49793 11 days ago |
99-54802 3 months ago |
0-0 0 seconds |
| 31571 |
erdOne author:erdOne |
feat(RingTheory): existence of local algebra with given residue field |
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
awaiting-author
|
225/0 |
Mathlib.lean,Mathlib/RingTheory/LocalRing/SeparableResidueField.lean |
2 |
7 |
['chrisflav', 'github-actions', 'jcommelin', 'mathlib4-merge-conflict-bot'] |
chrisflav assignee:chrisflav |
11-39950 11 days ago |
11-43407 11 days ago |
9-73319 9 days |
| 31176 |
mcdoll author:mcdoll |
feat(Analysis): Taylor's theorem with the integral remainder |
---
[](https://gitpod.io/from-referrer/)
|
t-analysis
awaiting-author
|
169/2 |
Mathlib.lean,Mathlib/Analysis/Calculus/TaylorIntegral.lean,Mathlib/Analysis/Normed/Operator/BoundedLinearMaps.lean,docs/100.yaml,docs/undergrad.yaml |
5 |
5 |
['github-actions', 'mathlib4-merge-conflict-bot', 'sgouezel'] |
sgouezel assignee:sgouezel |
10-83815 10 days ago |
10-83815 10 days ago |
7-32435 7 days |
| 30350 |
joelriou author:joelriou |
feat(AlgebraicGeometry): the pseudofunctor which sends a scheme to its category of sheaves of modules |
We define `Scheme.Modules.pseudofunctor : Pseudofunctor (LocallyDiscrete Schemeᵒᵖ) (Adj Cat)` which sends a scheme `X` to the category `X.Modules` of sheaves of modules (not to be be confused with the full subcategory of quasi-coherent sheaves). The target bicategory is the bicategory of adjunctions in the bicategory of categories: this means that we formalise both the pushforward and the pullback of sheaves of modules over schemes.
---
We should wait for #31807
- [x] depends on: #30335
- [x] depends on: #30318
- [x] depends on: #30342
[](https://gitpod.io/from-referrer/)
|
t-algebraic-geometry
awaiting-author
|
303/17 |
Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Sheaf/Abelian.lean,Mathlib/Algebra/Category/ModuleCat/Sheaf/PullbackContinuous.lean,Mathlib/AlgebraicGeometry/Modules/Sheaf.lean,Mathlib/CategoryTheory/Adjunction/CompositionIso.lean,Mathlib/CategoryTheory/Bicategory/Adjunction/Basic.lean,Mathlib/CategoryTheory/Bicategory/Adjunction/Cat.lean,Mathlib/CategoryTheory/Category/Cat.lean,Mathlib/Topology/Sheaves/SheafCondition/Sites.lean |
9 |
10 |
['erdOne', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
10-77233 10 days ago |
13-78839 13 days ago |
0-10715 2 hours |
| 30432 |
kckennylau author:kckennylau |
feat(AlgebraicGeometry): define the non-vanishing locus of a set in Proj |
Given a subset `s : Set A`, the non-vanishing locus of `s` is the set of points whose corresponding prime ideal does not fully contain `s`. In other words, where not all elements of `s` vanish.
I could not find a name for this in the literature.
---
[](https://gitpod.io/from-referrer/)
|
t-algebraic-geometry
awaiting-author
|
66/0 |
Mathlib/AlgebraicGeometry/ProjectiveSpectrum/Basic.lean |
1 |
4 |
['github-actions', 'jcommelin'] |
alexjbest assignee:alexjbest |
10-72931 10 days ago |
10-72931 10 days ago |
44-12068 44 days |
| 31984 |
kim-em author:kim-em |
feat: proposed definition of `ConvexSpace` |
Trying to get the ball rolling the notion of a space with convex combinations, I suggest:
```
class ConvexSpace (R : Type u) (M : Type v)
[PartialOrder R] [Semiring R] [IsStrictOrderedRing R] where
/-- Take a convex combination of a family of points with the given probability distribution. -/
convexCombination {ι : Type v} (f : FiniteProbability R ι) (xs : ι → M) : M
/-- Associativity of convex combination. -/
assoc
{κ : Type v} (f₀ : FiniteProbability R κ)
{ι : κ → Type v} (f₁ : (k : κ) → FiniteProbability R (ι k))
(xs : (k : κ) → (ι k) → M) :
convexCombination f₀ (fun m => convexCombination (f₁ m) (xs m)) =
convexCombination (f₀.comp f₁) (fun ⟨k, i⟩ => xs k i)
/-- A convex combination of a single point is that point. -/
single {ι : Type v} (i : ι) (x : M) : convexCombination (.single i) (fun _ => x) = x
/-- Convex combinations are determined by the points with non-zero weights. -/
-- Perhaps this follows from `assoc`, but I don't see how.
ext {ι : Type v} (f : FiniteProbability R ι) (xs xs' : ι → M)
(h : ∀ i, i ∈ f.support → xs i = xs' i) : convexCombination f xs = convexCombination f xs'
```
where
```
structure FiniteProbability (R : Type u) [LE R] [AddCommMonoid R] [One R] (ι : Type v)
extends weights : ι →₀ R where
/-- All weights are non-negative. -/
nonneg : ∀ m, 0 ≤ weights m
/-- The weights sum to 1. -/
total : weights.sum (fun _ r => r) = 1
```
The file also contains some TODOs for next steps. |
t-algebra label:t-algebra$ |
143/0 |
Mathlib.lean,Mathlib/LinearAlgebra/ConvexSpace.lean |
2 |
21 |
['ADedecker', 'github-actions', 'kim-em', 'plp127'] |
YaelDillies assignee:YaelDillies |
10-69357 10 days ago |
12-16950 12 days ago |
12-16990 12 days |
| 31989 |
Thmoas-Guan author:Thmoas-Guan |
feat(RingTheory): add ideal fg of Noetherian lemma |
In this PR, we added lemma `Ideal.FG.of_isNoetherianRing`.
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
easy
awaiting-author
|
4/0 |
Mathlib/RingTheory/Noetherian/Defs.lean |
1 |
8 |
['Thmoas-Guan', 'chrisflav', 'erdOne', 'github-actions', 'ocfnash'] |
nobody |
10-50854 10 days ago |
10-59450 10 days ago |
1-26232 1 day |
| 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 |
13 |
['AntoineChambert-Loir', 'erdOne', 'github-actions'] |
nobody |
10-43511 10 days ago |
174-82349 5 months ago |
0-33 33 seconds |
| 26975 |
Whysoserioushah author:Whysoserioushah |
feat: a norm_num extension for complex numbers |
co-authored-by : @thefundamentaltheor3m, @hrmacbeth
---
[](https://gitpod.io/from-referrer/)
|
t-meta |
394/12 |
Mathlib/Analysis/RCLike/Basic.lean,Mathlib/Tactic/NormNum/Eq.lean,Mathlib/Tactic/NormNum/NormNumI.lean,Mathlib/Tactic/NormNum/Result.lean,MathlibTest/norm_numI.lean |
5 |
54 |
['JovanGerb', 'Whysoserioushah', 'dupuisf', 'eric-wieser', 'github-actions', 'hrmacbeth', 'mathlib4-merge-conflict-bot'] |
nobody |
10-37246 10 days ago |
10-37261 10 days ago |
135-3976 135 days |
| 31817 |
kckennylau author:kckennylau |
chore: remove extra monic hypotheses from divByMonic and modByMonic lemmas |
---
[Zulip discussion](https://leanprover.zulipchat.com/#narrow/channel/217875-Is-there-code-for-X.3F/topic/modByMonic_add_div/with/556964888)
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
t-algebra
awaiting-author
label:t-algebra$ |
85/88 |
Mathlib/Algebra/Polynomial/CoeffMem.lean,Mathlib/Algebra/Polynomial/Div.lean,Mathlib/Algebra/Polynomial/FieldDivision.lean,Mathlib/Algebra/Polynomial/PartialFractions.lean,Mathlib/Algebra/Polynomial/RingDivision.lean,Mathlib/FieldTheory/Minpoly/Basic.lean,Mathlib/FieldTheory/Minpoly/Field.lean,Mathlib/FieldTheory/Minpoly/IsIntegrallyClosed.lean,Mathlib/LinearAlgebra/Charpoly/Basic.lean,Mathlib/LinearAlgebra/Matrix/Charpoly/Coeff.lean,Mathlib/RingTheory/Adjoin/PowerBasis.lean,Mathlib/RingTheory/AdjoinRoot.lean,Mathlib/RingTheory/IntegralClosure/IsIntegral/Basic.lean,Mathlib/RingTheory/IntegralDomain.lean,Mathlib/RingTheory/IsAdjoinRoot.lean,Mathlib/RingTheory/Polynomial/Eisenstein/IsIntegral.lean,Mathlib/RingTheory/Polynomial/Nilpotent.lean,Mathlib/RingTheory/PowerBasis.lean,Mathlib/RingTheory/PowerSeries/WeierstrassPreparation.lean,Mathlib/RingTheory/Spectrum/Prime/ChevalleyComplexity.lean |
20 |
19 |
['artie2000', 'bryangingechen', 'github-actions', 'jcommelin', 'kbuzzard', 'kckennylau', 'mathlib-bors'] |
jcommelin assignee:jcommelin |
10-34329 10 days ago |
10-72785 10 days ago |
4-37368 4 days |
| 30995 |
kckennylau author:kckennylau |
feat(RingTheory): replace ofLinearEquiv with limit |
For an `I`-adically complete `M` we define `limit : AdicCompletion I M ≃ₗ[R] M`. This replaces the existing `ofLinearEquiv : M ≃ₗ[R] AdicCompletion I M` which goes in the opposite direction, and should make #30989 and subsequent PR's smoother. It is intended to be used together with [AdicCompletion.mk](https://leanprover-community.github.io/mathlib4_docs/Mathlib/RingTheory/AdicCompletion/Basic.html#AdicCompletion.mk) : `AdicCompletion.AdicCauchySequence I M →ₗ[R] AdicCompletion I M`.
We also introduce `adicExpansion (ϖ : R) (hϖ : ϖ ∈ I) : (ℕ → M) →ₗ[R] AdicCauchySequence I M`, which sends a sequence `a : ℕ → M` to the Cauchy sequence `∑ ϖ ^ i • a i`.
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
awaiting-author
|
77/49 |
Mathlib/RingTheory/AdicCompletion/Algebra.lean,Mathlib/RingTheory/AdicCompletion/Basic.lean,Mathlib/RingTheory/AdicCompletion/RingHom.lean |
3 |
8 |
['erdOne', 'github-actions', 'jjdishere', 'kckennylau', 'mathlib4-merge-conflict-bot'] |
erdOne assignee:erdOne |
10-3149 10 days ago |
12-32234 12 days ago |
13-36353 13 days |
| 30620 |
plp127 author:plp127 |
feat: copy LE and LT on preorder and partial order |
Adds `Preorder.copy` and `PartialOrder.copy` for replacing the le and lt with provably equal ones.
---
[](https://gitpod.io/from-referrer/)
|
t-order
awaiting-author
|
22/0 |
Mathlib/Order/Defs/PartialOrder.lean |
1 |
6 |
['Vierkantor', 'github-actions', 'plp127'] |
Vierkantor assignee:Vierkantor |
9-77024 9 days ago |
9-77024 9 days ago |
31-54617 31 days |
| 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/)
---
- [ ] depends on: #23831
*This PR continues the work from #21693.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/21693* |
t-analysis
awaiting-author
|
37/0 |
Mathlib/Analysis/Analytic/Binomial.lean |
1 |
7 |
['erdOne', 'github-actions', 'j-loreaux', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'vasnesterov'] |
nobody |
9-76855 9 days ago |
9-79360 9 days ago |
8-29520 8 days |
| 32094 |
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.
---
I'm not happy about one detail:
- many options take an `Array String`: how can I pass this to the executable? This is not obvious to me...
- TODO: address the comment at https://github.com/leanprover-community/mathlib4/pull/14654#discussion_r1685824917
Continuation of #14654. Proof-of-concept; the real implementation should be in batteries/a separate repository.
---
[](https://gitpod.io/from-referrer/)
|
t-linter
CI
|
154/0 |
lakefile.lean,scripts/run_linter.lean |
2 |
1 |
['github-actions'] |
nobody |
9-74021 9 days ago |
9-74021 9 days ago |
9-74064 9 days |
| 31366 |
FaffyWaffles author:FaffyWaffles |
feat(Analysis/SpecialFunctions/StirlingRobbins): Robbins' sharp stepwise bound for stirlingSeq |
Introduces `Mathlib.Analysis.SpecialFunctions.StirlingRobbins`,
proving Robbins' sharp stepwise bound for the Stirling sequence.
* Main theorem: `log_stirlingSeq_diff_le`
* Improves the existing bound `1/(4k^2)` to the sharp `1/(12k(k+1))`
* Adds helper lemmas on summability and geometric bounds
* Complements `Stirling.lean`
References:
- https://leanprover-community.github.io/mathlib4_docs/Mathlib/Analysis/SpecialFunctions/Stirling.html
- Robbins (1955), *A Remark on Stirling’s Formula*
---
**Note for Transparency:** Assistance provided by AI tools (Claude and Aristotle) for drafting, text, and structure.
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-analysis
awaiting-author
|
64/5 |
Mathlib/Analysis/SpecialFunctions/Stirling.lean |
1 |
15 |
['FaffyWaffles', 'github-actions', 'j-loreaux', 'mathlib4-merge-conflict-bot', 'tb65536'] |
nobody |
9-37502 9 days ago |
9-37502 9 days ago |
4-57241 4 days |
| 31960 |
urkud author:urkud |
feat: a lower bound for the volume of a cone on the unit sphere |
---
- [x] depends on: #31956
- [x] depends on: #31957
[](https://gitpod.io/from-referrer/)
|
t-measure-probability |
95/0 |
Mathlib/MeasureTheory/Constructions/HaarToSphere.lean |
1 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
kim-em assignee:kim-em |
9-26020 9 days ago |
9-39031 9 days ago |
9-41579 9 days |
| 31796 |
dobronx1325 author:dobronx1325 |
feat(Data/Real/EReal): add mul_lt_mul_of_pos_left theorem |
This PR adds the theorem `EReal.mul_lt_mul_of_pos_left`, which states that for a positive real number `a` and extended reals `b < c`, left multiplication by `a` preserves the strict order: `(a : EReal) * b < (a : EReal) * c`.
The theorem complements existing order-preserving properties for addition in `EReal` and extends the algebraic structure for multiplication. The proof uses basic properties of extended reals and order relations.
---
[](https://gitpod.io/from-referrer/)
|
t-data
new-contributor
|
23/0 |
Mathlib/Data/EReal/Operations.lean |
1 |
4 |
['JovanGerb', 'LLaurance', 'dobronx1325', 'github-actions'] |
nobody |
9-15808 9 days ago |
16-10531 16 days ago |
16-10571 16 days |
| 26743 |
grunweg author:grunweg |
feat: 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
|
200/23 |
Mathlib/Geometry/Manifold/VectorField/LieBracket.lean,Mathlib/Geometry/Manifold/VectorField/Pullback.lean |
2 |
3 |
['github-actions', 'grunweg', 'mathlib4-merge-conflict-bot'] |
nobody |
8-81117 8 days ago |
8-82221 8 days ago |
0-1 1 second |
| 31210 |
jsm28 author:jsm28 |
feat(Geometry/Euclidean/MongePoint): `reindex` lemmas |
Add lemmas about `mongePoint`, `mongePlane` and `orthocenter` applied to `Simplex.reindex`.
---
[](https://gitpod.io/from-referrer/)
|
t-euclidean-geometry |
28/0 |
Mathlib/Geometry/Euclidean/MongePoint.lean |
1 |
4 |
['JovanGerb', 'github-actions', 'jsm28'] |
JovanGerb assignee:JovanGerb |
8-72815 8 days ago |
32-21907 1 month ago |
32-21885 32 days |
| 27258 |
JovanGerb author:JovanGerb |
feat: 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.
---
- [x] depends on: #27257
[](https://gitpod.io/from-referrer/)
|
IMO
awaiting-author
|
335/0 |
Archive.lean,Archive/Imo/Imo2020Q6.lean |
2 |
14 |
['JovanGerb', 'dwrensha', 'github-actions', 'jsm28', 'mathlib4-dependent-issues-bot'] |
dwrensha assignee:dwrensha |
8-67486 8 days ago |
8-67486 8 days ago |
64-78344 64 days |
| 31362 |
BeibeiX0 author:BeibeiX0 |
feat(partitions): generalized pentagonal numbers |
feat(partitions): generalized pentagonal numbers and error term eₙ
Introduce infrastructure around Euler’s pentagonal number theorem:
* Define parity counters for strict partitions:
- `p_even_distinct n`
- `p_odd_distinct n`
- `strict_partitions_parity_diff n := (p_even_distinct n : ℤ) - (p_odd_distinct n : ℤ)`
* Generalized pentagonal numbers:
- `generalizedPentagonalZ : ℤ → ℤ` with basic API (`gpn_nonneg`, `gpn_coe`)
- `generalizedPentagonalNum : ℤ → ℕ`
- parity lemma `even_neg_j_add_three_j_sq` and `even_neg_j_add_three_j_sq'`
- search window equivalence `exists_j_iff_exists_j_in_range`
- `Decidable (∃ j : ℤ, n = generalizedPentagonalZ j)` via a bounded range
* Euler error term:
- `error_term_e n : ℤ` (≔ `(-1)^{|j|}` if `n = generalizedPentagonalZ j` for some `j`,
and `0` otherwise)
* Finite product cut-off of the generating function:
- `E n : PowerSeries ℤ := ∏_{k=1}^{n+1} (1 - X^k)`
- lemma `coeff_E_eq_coeff_cutoff`
Implementation notes:
* Keep the integer-valued version `generalizedPentagonalZ` for arithmetic lemmas and
signs; obtain the natural-number version via `Int.toNat`.
* The bounded search lemma gives a small window `j ∈ [-(n+1), n+1]` for decidability.
Motivation:
* This is groundwork for proofs of Euler’s pentagonal number theorem and parity
identities relating strict partitions to the error term.
References:
* https://en.wikipedia.org/wiki/Pentagonal_number_theorem |
new-contributor
t-combinatorics
awaiting-author
|
258/0 |
Mathlib.lean,Mathlib/Combinatorics/Enumerative/PentagonalNumbers.lean |
2 |
8 |
['BeibeiX0', 'dagurtomas', 'github-actions', 'mathlib4-merge-conflict-bot', 'wwylele'] |
awainverse assignee:awainverse |
8-64722 8 days ago |
8-64722 8 days ago |
15-20162 15 days |
| 31755 |
kaantahti author:kaantahti |
feat(Combinatorics): Add Sperner's Lemma formalization |
Complete formalization of Sperner's Lemma with rigorous proofs:
- Main theorems: strong_sperner (odd count) and sperner (existence)
- 13 fully proven auxiliary lemmas
- 8 documented axioms for simplicial complex API
- ~750 lines, zero sorries
- Addresses issue #25231
This formalization proves both the strong version (odd number of panchromatic faces) and the existence version of Sperner's Lemma. The proof uses induction on dimension with a complete parity argument via boundary counting.
The 8 axioms represent standard results from simplicial complex theory that are currently missing from mathlib4's geometric API. Each axiom is documented with mathematical justification and difficulty rating.
Closes #25231
|
new-contributor
t-combinatorics
WIP
|
7725/0 |
Mathlib.lean,Mathlib/Analysis/Convex/SimplicialComplex/Boundary.lean,Mathlib/Combinatorics/Sperner.lean,PR_COMMENT_DRAFT.md |
4 |
4 |
['LLaurance', 'github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
8-64095 8 days ago |
8-64095 8 days ago |
8-13311 8 days |
| 30030 |
JonBannon author:JonBannon |
feat(MeasureTheory): add `MemLp.Const` class and instances to unify `p = ∞` and `μ.IsFiniteMeasure` cases |
Although it is possible to ensure that, for example, the `One` instances for `p=∞` and `μ.IsFiniteMeasure` are defeq, introducing an `MemLp.Const` typeclass removes the need to unfold extensively to check this definitional equality, improving performance. cf. https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Lp.20constant.20function.20issue/with/537563137
This PR introduces the requisite class and associated instances.
---
[](https://gitpod.io/from-referrer/)
|
t-measure-probability
awaiting-author
|
224/137 |
Mathlib/MeasureTheory/Function/ConditionalExpectation/AEMeasurable.lean,Mathlib/MeasureTheory/Function/ContinuousMapDense.lean,Mathlib/MeasureTheory/Function/L1Space/Integrable.lean,Mathlib/MeasureTheory/Function/LocallyIntegrable.lean,Mathlib/MeasureTheory/Function/LpSeminorm/Basic.lean,Mathlib/MeasureTheory/Function/LpSpace/Basic.lean,Mathlib/MeasureTheory/Function/LpSpace/ContinuousCompMeasurePreserving.lean,Mathlib/MeasureTheory/Function/LpSpace/DomAct/Basic.lean,Mathlib/MeasureTheory/Function/LpSpace/Indicator.lean,Mathlib/MeasureTheory/Function/SimpleFuncDenseLp.lean,Mathlib/MeasureTheory/Integral/IntegrableOn.lean,Mathlib/MeasureTheory/Integral/SetToL1.lean,Mathlib/MeasureTheory/Measure/SeparableMeasure.lean |
13 |
24 |
['JonBannon', 'github-actions', 'j-loreaux', 'mathlib4-merge-conflict-bot'] |
urkud assignee:urkud |
8-63274 8 days ago |
14-64653 14 days ago |
19-64975 19 days |
| 31315 |
Parcly-Taxel author:Parcly-Taxel |
feat: IMO 2010 Q5 |
I use an opaque power function to avoid `(kernel) deep recursion detected`. Cf. [#general > Panic in rw: Nat.pow exponent is too big @ 💬](https://leanprover.zulipchat.com/#narrow/channel/113488-general/topic/Panic.20in.20rw.3A.20Nat.2Epow.20exponent.20is.20too.20big/near/513294906). |
IMO
awaiting-author
|
252/0 |
Archive.lean,Archive/Imo/Imo2010Q5.lean |
2 |
2 |
['github-actions', 'jsm28'] |
dwrensha assignee:dwrensha |
8-63238 8 days ago |
8-63238 8 days ago |
20-37914 20 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
- [x] depends on: #30287
[](https://gitpod.io/from-referrer/)
|
t-combinatorics
awaiting-author
|
117/7 |
Mathlib/Combinatorics/SimpleGraph/CompleteMultipartite.lean |
1 |
26 |
['YaelDillies', 'b-mehta', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'mitchell-horner'] |
YaelDillies assignee:YaelDillies |
8-63185 8 days ago |
8-63185 8 days ago |
56-71462 56 days |
| 31592 |
gasparattila author:gasparattila |
chore(Tactic/Measurability): `fun_prop` lemmas for solving `MeasurableSet {x | ...}` goals |
Currently, lemmas of the form `MeasurableSet {x | ...}` cannot be used by `measurability`, because `simp` changes the goal to `Measurable fun x => ...`. This PR adds the necessary `fun_prop` lemmas so that they work with `measurability` (except for statements involving equality, which are done in #31512). This fixes #26620.
---
[](https://gitpod.io/from-referrer/)
|
t-measure-probability |
21/7 |
Mathlib/MeasureTheory/Constructions/BorelSpace/Order.lean,Mathlib/MeasureTheory/MeasurableSpace/Constructions.lean,MathlibTest/measurability.lean |
3 |
7 |
['ADedecker', 'gasparattila', 'github-actions'] |
kex-y assignee:kex-y |
8-37748 8 days ago |
21-65736 21 days ago |
21-65776 21 days |
| 30744 |
grunweg author:grunweg |
feat: more extensions for differential geometry elaborators |
Support inferring a model with corners in all remaining instances in mathlib, except for products and direct sums:
- on Euclidean space, half-space or quadrants.
- for the units in a normed algebra (including GL(V))
- the unit interval
- on the complex unit circle
- on a metric sphere in a real or complex inner product space (WIP)
---
- [x] depends on: #30413
- [x] depends on: #30879
[](https://gitpod.io/from-referrer/)
|
t-differential-geometry
t-meta
|
487/32 |
Mathlib/Geometry/Manifold/Instances/UnitsOfNormedAlgebra.lean,Mathlib/Geometry/Manifold/Notation.lean,MathlibTest/DifferentialGeometry/Notation.lean,MathlibTest/DifferentialGeometry/NotationAdvanced.lean |
4 |
10 |
['github-actions', 'grunweg', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'thorimur'] |
thorimur assignee:thorimur |
8-28448 8 days ago |
8-77028 8 days ago |
8-79607 8 days |
| 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.
---
- [x] depends on: #29503
- [x] depends on: #29507
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-measure-probability
awaiting-author
|
673/9 |
Mathlib.lean,Mathlib/Algebra/BigOperators/Group/Finset/Gaps.lean,Mathlib/Analysis/Analytic/OfScalars.lean,Mathlib/Analysis/Real/OfDigits.lean,Mathlib/MeasureTheory/Covering/Vitali.lean,Mathlib/MeasureTheory/Function/AbsolutelyContinuous.lean,Mathlib/MeasureTheory/Integral/IntervalIntegral/AbsContFunc.lean,Mathlib/MeasureTheory/Integral/IntervalIntegral/Basic.lean,Mathlib/Order/Interval/Finset/Gaps.lean,Mathlib/Topology/Algebra/InfiniteSum/Basic.lean,Mathlib/Topology/Algebra/InfiniteSum/Real.lean |
11 |
6 |
['github-actions', 'jcommelin', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'zhuyizheng'] |
sgouezel assignee:sgouezel |
8-28082 8 days ago |
8-59402 8 days ago |
2-7960 2 days |
| 30293 |
vlad902 author:vlad902 |
feat(SimpleGraph): there exists a maximal path/trail in a graph with finite edges |
Inspired by [this Zulip thread](https://leanprover.zulipchat.com/#narrow/channel/252551-graph-theory/topic/Help.20me.20learn.20good.20style.3A.20IsTree/near/543395218)
---
[](https://gitpod.io/from-referrer/)
|
t-combinatorics |
29/0 |
Mathlib/Combinatorics/SimpleGraph/Paths.lean |
1 |
5 |
['SnirBroshi', 'github-actions', 'mathlib4-merge-conflict-bot', 'vlad902'] |
awainverse assignee:awainverse |
8-27268 8 days ago |
8-38360 8 days ago |
54-43388 54 days |
| 30886 |
urkud author:urkud |
feat(DifferentialForm): exterior derivative applied to vector fields |
---
- [ ] depends on: #30331
[](https://gitpod.io/from-referrer/)
|
t-analysis |
217/0 |
Mathlib.lean,Mathlib/Analysis/Calculus/DifferentialForm/VectorField.lean,Mathlib/Analysis/Calculus/FDeriv/ContinuousAlternatingMap.lean,Mathlib/Topology/Algebra/Module/Alternating/Basic.lean |
4 |
4 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
kex-y assignee:kex-y |
8-26020 8 days ago |
9-38987 9 days ago |
18-7452 18 days |
| 30525 |
515801431 author:515801431 |
feat(Mathlib/Combinatorics/Enumerative/Polya): Add Polya Counting |
This PR introduces basic definitions and results about colorings under permutation group actions.
A coloring is defined as a function X → Y, and the permutation group Equiv.Perm X acts on colorings by precomposition:
(g • c) x = c (g⁻¹ • x)
This formalizes the natural action of relabeling the elements of X.
Main definitions
MulAction (Equiv.Perm X) (X → Y):
The action of the permutation group on colorings via precomposition.
coloringEquiv (c₁ c₂ : X → Y) : Prop:
Two colorings are equivalent if they lie in the same orbit under this action, i.e.
∃ f : Equiv.Perm X, f • c₁ = c₂.
Main results
smul_eq_iff_mem_stabilizer:
Characterizes when two group actions on the same coloring are equal, showing that
g • c = f • c ↔ f⁻¹ * g ∈ stabilizer c.
coloringEquiv_equivalence:
Proves that coloringEquiv defines an equivalence relation on X → Y.
orbit_size_eq_index:
Reformulates the orbit–stabilizer theorem in the context of colorings:
|orbit c| = |Perm X| / |stabilizer c|
Motivation
These results provide foundational infrastructure for studying Burnside’s lemma and Pólya’s enumeration theorem in Mathlib, where the enumeration of distinct colorings up to symmetry plays a central role. |
new-contributor
t-combinatorics
awaiting-author
|
113/0 |
Mathlib.lean,Mathlib/Combinatorics/Enumerative/Polya.lean |
2 |
7 |
['IvanRenison', 'alreadydone', 'github-actions', 'mathlib4-merge-conflict-bot'] |
awainverse assignee:awainverse |
8-4470 8 days ago |
8-4470 8 days ago |
40-50241 40 days |
| 30750 |
SnirBroshi author:SnirBroshi |
feat(Data/Quot): `toSet` and `equivClassOf` |
Define `toSet` which gets the set corresponding to an element of a quotient, and `equivClassOf` which gets the equivalence class of an element under a quotient.
---
I found these definitions helpful when working with quotients, specifically `ConnectedComponents` of a `TopologicalSpace`.
Additionally, I need `equivSigmaToSet` (in `Data/Setoid/Basic`) to prove things about `SimpleGraph.ConnectedComponent`.
[](https://gitpod.io/from-referrer/)
|
t-data
awaiting-zulip
awaiting-author
|
179/0 |
Mathlib/Data/Quot.lean,Mathlib/Data/Set/Image.lean,Mathlib/Data/SetLike/Basic.lean,Mathlib/Data/Setoid/Basic.lean |
4 |
3 |
['TwoFX', 'eric-wieser', 'github-actions'] |
TwoFX assignee:TwoFX |
8-1006 8 days ago |
8-1006 8 days ago |
36-69524 36 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
---
- [x] depends on: #29594
- [x] depends on: #29644
[](https://gitpod.io/from-referrer/)
|
t-order
t-algebra
label:t-algebra$ |
113/2 |
Mathlib/Algebra/GroupWithZero/Range.lean,Mathlib/Algebra/Order/GroupWithZero/Range.lean |
2 |
109 |
['YaelDillies', 'eric-wieser', 'faenuccio', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'pechersky'] |
YaelDillies assignee:YaelDillies |
8-1 8 days ago |
8-25 7 days ago |
64-4942 64 days |
| 31579 |
xroblot author:xroblot |
feat(Data/Nat/Digits): prove the bijection induced by `Nat.ofDigits` and use it to compute the sum of the sum of digits |
We prove that `Nat.ofDigits` induces a bijection between the set of list of natural integers of length `l`
with coefficients `< b` and the set of natural integers `< b ^ l` and develop some API.
As a application, we prove that
```lean
theorem Nat.sum_digits_sum_eq {b : ℕ} (hb : 1 < b) (l : ℕ) :
∑ x ∈ Finset.range (b ^ l), (b.digits x).sum = l * b ^ (l - 1) * b.choose 2
```
---
|
t-data |
189/0 |
Mathlib/Data/Nat/Digits/Lemmas.lean |
1 |
11 |
['TwoFX', 'eric-wieser', 'github-actions', 'mathlib4-merge-conflict-bot', 'xroblot'] |
TwoFX assignee:TwoFX |
7-70870 7 days ago |
7-70870 7 days ago |
21-67370 21 days |
| 32039 |
HugLycan author:HugLycan |
Feat/positivity-zeroness |
---
WIP...
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-meta
WIP
|
528/131 |
Mathlib/Tactic/Positivity/Basic.lean,Mathlib/Tactic/Positivity/Core.lean,Mathlib/Tactic/Positivity/test_Basic.lean |
3 |
2 |
['github-actions'] |
nobody |
7-66940 7 days ago |
7-66973 7 days ago |
0-16 16 seconds |
| 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.
`StarAlgEquiv` now extends `AlgEquiv`. We also generalize a few files to allow for non-unital.
I suspect there are a few more things to generalize, but will leave this for later.
Co-authored-by: Jireh Loreaux
---
Revives #8686.
[](https://gitpod.io/from-referrer/)
|
t-algebra
awaiting-author
label:t-algebra$ |
559/480 |
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/SkewMonoidAlgebra/Lift.lean,Mathlib/Algebra/Star/Free.lean,Mathlib/Algebra/Star/StarAlgHom.lean,Mathlib/Analysis/CStarAlgebra/Spectrum.lean,Mathlib/Analysis/Normed/Algebra/GelfandFormula.lean,Mathlib/Analysis/Normed/Algebra/Spectrum.lean,Mathlib/Analysis/Normed/Algebra/UnitizationL1.lean,Mathlib/Analysis/Normed/Lp/LpEquiv.lean,Mathlib/Analysis/Normed/Module/Basic.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/Notation.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/LinearAlgebra/TensorProduct/Subalgebra.lean,Mathlib/NumberTheory/NumberField/Cyclotomic/Ideal.lean,Mathlib/NumberTheory/NumberField/Discriminant/Defs.lean,Mathlib/RingTheory/AdicCompletion/Algebra.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/Maps.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 |
101 |
61 |
['fpvandoorn', 'github-actions', 'jcommelin', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'leanprover-radar', 'mathlib4-merge-conflict-bot', 'themathqueen'] |
joelriou assignee:joelriou |
7-64816 7 days ago |
8-35403 8 days ago |
69-64557 69 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
awaiting-author
label:t-algebra$ |
59/17 |
Mathlib/Algebra/Colimit/DirectLimit.lean,Mathlib/Algebra/Ring/Defs.lean,Mathlib/LinearAlgebra/CliffordAlgebra/Basic.lean |
3 |
26 |
['alreadydone', 'github-actions', 'j-loreaux', 'kckennylau', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'riccardobrasca'] |
riccardobrasca assignee:riccardobrasca |
7-59323 7 days ago |
7-59323 7 days ago |
57-29954 57 days |
| 27053 |
tb65536 author:tb65536 |
feat: Galois group of `x^n - x - 1` |
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebra
WIP
label:t-algebra$ |
357/7 |
Mathlib/RingTheory/Polynomial/Selmer.lean |
1 |
6 |
['AntoineChambert-Loir', 'github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
7-52110 7 days ago |
7-52118 7 days ago |
0-1 1 second |
| 31500 |
zcyemi author:zcyemi |
feat(Analysis/Convex/Between): add lemmas on affine independence under strict betweenness |
---
Add lemmas showing that affine independence is preserved when replacing a vertex
by a point strictly between two others, and related results for triangles.
deps:
- [ ] depends on: #31498
- [ ] depends on: #31499
|
t-convex-geometry
awaiting-author
|
101/0 |
Mathlib/Analysis/Convex/Between.lean,Mathlib/LinearAlgebra/AffineSpace/FiniteDimensional.lean,Mathlib/LinearAlgebra/AffineSpace/Independent.lean |
3 |
5 |
['github-actions', 'mathlib4-dependent-issues-bot', 'ocfnash', 'zcyemi'] |
nobody |
7-51765 7 days ago |
7-51765 7 days ago |
7-39716 7 days |
| 32186 |
urkud author:urkud |
feat(Integral): estimate displacement by the integral of the speed |
This PR adds yet another form of the Mean Value Theorem. I don't know if we can refactor the proofs to reduce code duplication. I'll add more versions before marking the PR as ready for review.
---
[](https://gitpod.io/from-referrer/)
|
t-measure-probability |
81/0 |
Mathlib.lean,Mathlib/MeasureTheory/Integral/IntervalIntegral/DistLEIntegral.lean |
2 |
1 |
['github-actions'] |
nobody |
7-44702 7 days ago |
7-44709 7 days ago |
0-0 0 seconds |
| 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.
---
- [x] depends on: #26457
- [x] depends on: #26282
- [x] depends on: #26281
- [x] depends on: #26280
- [x] depends on: #26279
[](https://gitpod.io/from-referrer/)
|
t-group-theory |
548/20 |
Mathlib.lean,Mathlib/GroupTheory/GroupAction/MultiplePrimitivity.lean,Mathlib/GroupTheory/GroupAction/MultipleTransitivity.lean,Mathlib/GroupTheory/Perm/MaximalSubgroups.lean,Mathlib/GroupTheory/SpecificGroups/Alternating.lean,Mathlib/GroupTheory/SpecificGroups/Alternating/MaximalSubgroups.lean |
6 |
n/a |
['AntoineChambert-Loir', 'adomani', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
7-37611 7 days ago |
unknown |
unknown |
| 31062 |
zcyemi author:zcyemi |
feat(Geometry/Euclidean/Similarity): add triangle similarity |
---
Add theorems about similarity of triangles.
[](https://gitpod.io/from-referrer/)
|
t-euclidean-geometry
awaiting-author
|
279/0 |
Mathlib.lean,Mathlib/Geometry/Euclidean/Similarity.lean,Mathlib/Topology/MetricSpace/Similarity.lean |
3 |
26 |
['github-actions', 'jsm28', 'mathlib4-merge-conflict-bot', 'zcyemi'] |
jsm28 assignee:jsm28 |
7-28547 7 days ago |
7-28547 7 days ago |
14-65902 14 days |
| 30344 |
Deep0Thinking author:Deep0Thinking |
feat(MeasureTheory/Integral): add versions of `exists_eq_interval_average` and first mean value theorem for integrals |
Add the First mean value theorem for (unordered) interval integrals on ℝ.
- `exists_eq_const_mul_interval_integral_of_continuous_on_of_ae_nonneg`
- `exists_eq_const_mul_interval_integral_of_continuous_on_of_nonneg`
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-measure-probability
|
294/41 |
Mathlib.lean,Mathlib/MeasureTheory/Integral/IntervalAverage.lean,Mathlib/MeasureTheory/Integral/IntervalIntegral/MeanValue.lean |
3 |
10 |
['Deep0Thinking', 'github-actions', 'mathlib4-merge-conflict-bot', 'plp127'] |
kex-y assignee:kex-y |
7-26037 7 days ago |
10-41223 10 days ago |
51-84560 51 days |
| 31979 |
jsm28 author:jsm28 |
feat(LinearAlgebra/AffineSpace/Independent): injectivity of spans of images |
Add the lemma
```lean
lemma AffineIndependent.injective_affineSpan_image [Nontrivial k] {p : ι → P}
(ha : AffineIndependent k p) : Injective fun (s : Set ι) ↦ affineSpan k (p '' s) := by
```
which is straightforward given existing lemmas, and the corresponding `vectorSpan` lemma
```lean
lemma AffineIndependent.vectorSpan_image_eq_iff [Nontrivial k] {p : ι → P}
(ha : AffineIndependent k p) {s₁ s₂ : Set ι} :
vectorSpan k (p '' s₁) = vectorSpan k (p '' s₂) ↔
s₁ = s₂ ∨ s₁.Subsingleton ∧ s₂.Subsingleton := by
```
(feel free to golf).
---
- [ ] depends on: #31978
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
76/0 |
Mathlib/LinearAlgebra/AffineSpace/Independent.lean |
1 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
kim-em assignee:kim-em |
7-26026 7 days ago |
10-49883 10 days ago |
10-50553 10 days |
| 32041 |
thomaskwaring author:thomaskwaring |
feat(Combinatorics/SimpleGraph/Acyclic): every acyclic subgraph can be extended to a maximal one |
We show that every acyclic subgraph can be extended to a maximal acyclic subgraph.
--- |
new-contributor
t-combinatorics
|
32/0 |
Mathlib/Combinatorics/SimpleGraph/Acyclic.lean |
1 |
1 |
['github-actions'] |
kmill assignee:kmill |
7-26023 7 days ago |
10-80128 10 days ago |
10-80165 10 days |
| 32042 |
chrisflav author:chrisflav |
feat(AlgebraicGeometry): quasi compact covers |
This will be used to define the fpqc topology on `Scheme`.
From Proetale.
---
[](https://gitpod.io/from-referrer/)
|
t-algebraic-geometry |
311/1 |
Mathlib.lean,Mathlib/AlgebraicGeometry/Cover/QuasiCompact.lean,Mathlib/AlgebraicGeometry/Morphisms/Affine.lean,Mathlib/AlgebraicGeometry/Morphisms/QuasiCompact.lean,Mathlib/AlgebraicGeometry/Morphisms/UnderlyingMap.lean,Mathlib/AlgebraicGeometry/Sites/MorphismProperty.lean,Mathlib/Topology/Sets/CompactOpenCovered.lean,Mathlib/Topology/Spectral/Prespectral.lean |
8 |
9 |
['chrisflav', 'erdOne', 'github-actions'] |
joneugster assignee:joneugster |
7-26022 7 days ago |
10-79711 10 days ago |
10-79689 10 days |
| 31995 |
Thmoas-Guan author:Thmoas-Guan |
feat(RingTheory) : Module being injective is local property |
In this PR, we proved that for module over Noetherian ring, being injective is local property.
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
awaiting-author
|
235/0 |
Mathlib.lean,Mathlib/RingTheory/LocalProperties/Injective.lean |
2 |
4 |
['Thmoas-Guan', 'dagurtomas', 'github-actions'] |
nobody |
7-18311 7 days ago |
8-39910 8 days ago |
3-30007 3 days |
| 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`
---
- [x] depends on: #29882
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
awaiting-author
|
250/0 |
Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Baer.lean,Mathlib/RingTheory/GlobalDimension.lean |
3 |
13 |
['Thmoas-Guan', 'erdOne', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
erdOne assignee:erdOne |
7-13884 7 days ago |
14-86276 14 days ago |
27-39065 27 days |
| 31929 |
kim-em author:kim-em |
feat: replace `Finsupp.embDomain_apply` with more general lemma |
- [ ] depends on #31927
- [ ] depends on #31928 |
delegated |
24/22 |
Mathlib/Algebra/BigOperators/Finsupp/Basic.lean,Mathlib/Algebra/Polynomial/Reverse.lean,Mathlib/Analysis/Fourier/BoundedContinuousFunctionChar.lean,Mathlib/Data/Finsupp/Basic.lean,Mathlib/Data/Finsupp/Defs.lean,Mathlib/Data/Finsupp/Option.lean,Mathlib/Data/Finsupp/Sigma.lean,Mathlib/Data/Finsupp/Single.lean,Mathlib/Data/List/ToFinsupp.lean |
9 |
5 |
['eric-wieser', 'github-actions', 'jcommelin', 'mathlib-bors', 'mathlib4-merge-conflict-bot'] |
nobody |
7-13342 7 days ago |
7-13425 7 days ago |
2-51105 2 days |
| 32169 |
saodimao20 author:saodimao20 |
feat: add convolution_comp_add_right |
This PR adds a lemma `convolution_comp_translation_right` showing that convolution commutes with translation on the right operand. Specifically, it proves that for an additive commutative group $G$, the convolution of a function $f$ with a translated function $x \mapsto g(a + x)$ is equal to the convolution of $f$ and $g$ evaluated at $x + a$.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-analysis
awaiting-author
|
14/0 |
Mathlib/Analysis/Convolution.lean |
1 |
3 |
['github-actions', 'urkud'] |
nobody |
7-2188 7 days ago |
7-2188 7 days ago |
0-82278 22 hours |
| 31455 |
kim-em author:kim-em |
feat: products of locally contractible spaces |
---
- [x] depends on: #31453
- [x] depends on: #31454
Note: Proofs in this PR were developed with assistance from Claude. |
t-topology
delegated
|
31/10 |
Mathlib/Topology/Homotopy/LocallyContractible.lean |
1 |
7 |
['github-actions', 'j-loreaux', 'mathlib-bors', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'urkud'] |
dagurtomas assignee:dagurtomas |
7-1116 7 days ago |
9-6271 9 days ago |
9-58985 9 days |
| 31059 |
gasparattila author:gasparattila |
feat(Topology/Sets): define the Vietoris topology on `(Nonempty)Compacts` |
This PR defines the Vietoris topology on `Compacts` and `NonemptyCompacts`, and proves that it is induced by the Hausdorff uniformity.
---
- [x] depends on: #31031
- [x] depends on: #31058
[](https://gitpod.io/from-referrer/)
|
t-topology |
227/29 |
Mathlib.lean,Mathlib/Data/Rel.lean,Mathlib/Topology/MetricSpace/Closeds.lean,Mathlib/Topology/Sets/Compacts.lean,Mathlib/Topology/Sets/VietorisTopology.lean,Mathlib/Topology/UniformSpace/Closeds.lean |
6 |
6 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'robin-carlier'] |
ADedecker assignee:ADedecker |
6-84359 6 days ago |
6-84506 6 days ago |
14-17842 14 days |
| 31219 |
Thmoas-Guan author:Thmoas-Guan |
feat(Algebra): lemma about `IsBaseChange` under exact sequence |
In this lemma, we proved cokernel preserve `IsBaseChange S` and kernel preserve `IsBaseChange S` when `S` is flat.
Co-authored-by: Wang Jingting
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
awaiting-author
|
105/0 |
Mathlib.lean,Mathlib/RingTheory/Flat/IsBaseChange.lean |
2 |
8 |
['Thmoas-Guan', 'erdOne', 'github-actions', 'mathlib4-merge-conflict-bot', 'urkud'] |
nobody |
6-84075 6 days ago |
12-31796 12 days ago |
16-43808 16 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 |
215/180 |
Mathlib/Order/Hom/Basic.lean |
1 |
17 |
['YaelDillies', 'github-actions', 'linesthatinterlace', 'mathlib4-merge-conflict-bot'] |
b-mehta and linesthatinterlace assignee:b-mehta assignee:linesthatinterlace |
6-83963 6 days ago |
10-55951 10 days ago |
36-62055 36 days |
| 30133 |
smmercuri author:smmercuri |
feat: `WithVal v` and `WithVal w` are isomorphic as uniform spaces when `v` and `w` are equivalent valuations |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-topology
label:t-algebra$ |
101/0 |
Mathlib/Algebra/Order/Hom/Ring.lean,Mathlib/RingTheory/Valuation/Basic.lean,Mathlib/Topology/Algebra/Valued/WithVal.lean |
3 |
10 |
['github-actions', 'kbuzzard', 'kckennylau', 'robin-carlier', 'smmercuri'] |
kbuzzard and pechersky assignee:pechersky assignee:kbuzzard |
6-73563 6 days ago |
6-77707 6 days ago |
29-10093 29 days |
| 31132 |
kckennylau author:kckennylau |
feat(Algebra): saturation of a submonoid |
This PR defines the saturation of a submonoid and the type of saturated submonoids.
It is used for the context of localisations.
Caveat: there is a similarly named predicate called `AddSubgroup.Saturated`.
Zulip:
* [mathlib4 > saturation of a submonoid](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/saturation.20of.20a.20submonoid/with/548242862)
* [#Is there code for X? > Closure of Submonoid in CommMonoids](https://leanprover.zulipchat.com/#narrow/channel/217875-Is-there-code-for-X.3F/topic/Closure.20of.20Submonoid.20in.20CommMonoids/near/419087778)
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
278/0 |
Mathlib/Algebra/Group/Submonoid/Saturation.lean |
1 |
12 |
['github-actions', 'kckennylau', 'mathlib4-merge-conflict-bot', 'plp127'] |
kim-em assignee:kim-em |
6-72383 6 days ago |
14-70088 14 days ago |
33-21219 33 days |
| 31662 |
edwin1729 author:edwin1729 |
feat(Topology/Order): topological basis of scott topology on Complete… |
…PartialOrder
---
[Zulip discussion](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/.3E.20Algebraic.20complete.20partial.20order.20and.20domain.20theory/with/536359313) for this PR.
(1/2) PRs in domain theory, proving that scott topologies over Algebraic DCPOs (`CompletePartialOrder`) are sober.
The main reference is [Reneta, Duality in Domain Theory](https://alyata.github.io/documents/duality_domain_theory.pdf). But the statements can also be found in the canonical text [Abramsky and Jung](https://www.cs.ox.ac.uk/people/samson.abramsky/handbook.pdf)
This first PR proves two prerequisites, namely:
- the specialization order induced by the scott topology corresponds to the existing order of the DCPO. Prop 3.1.5 in [Duality in Domain Theory](https://alyata.github.io/documents/duality_domain_theory.pdf) and Prop 2.3.2(1) in [Abramsky and Jung](https://www.cs.ox.ac.uk/people/samson.abramsky/handbook.pdf)
- the upward closures of compact elements of the DCPO form a topological basis for the Scott Topology. Prop 3.5.2 in [Duality in Domain Theory](https://alyata.github.io/documents/duality_domain_theory.pdf) and Prop 2.3.6(2) in [Abramsky and Jung](https://www.cs.ox.ac.uk/people/samson.abramsky/handbook.pdf)
**The next PR is here:** #31670
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-topology
awaiting-author
|
293/1 |
Mathlib.lean,Mathlib/Topology/Order/ScottTopology.lean,Mathlib/Topology/Order/ScottTopologyDCPO.lean,docs/references.bib |
4 |
37 |
['b-mehta', 'edwin1729', 'github-actions', 'mathlib4-merge-conflict-bot', 'plp127'] |
b-mehta assignee:b-mehta |
6-68609 6 days ago |
6-68609 6 days ago |
12-62657 12 days |
| 28546 |
Sfgangloff author:Sfgangloff |
feat(SymbolicDynamics): basic setup of Zd, full shift, cylinders, pat… |
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
awaiting-author
|
751/0 |
Mathlib.lean,Mathlib/Dynamics/SymbolicDynamics/Basic.lean |
2 |
146 |
['Sfgangloff', 'eric-wieser', 'github-actions', 'kckennylau', 'mathlib4-merge-conflict-bot', 'sgouezel'] |
sgouezel assignee:sgouezel |
6-61383 6 days ago |
7-66137 7 days ago |
76-18097 76 days |
| 30892 |
vihdzp author:vihdzp |
feat: head/last element of flattened list |
---
Split off from #16837.
`Mathlib.Data.List.Induction` is not a heavy import by any sense of the word. The huge import jump seems to be artifact from the fact the file was previously importing only very minimal stuff from core. (In fact, the other theorems on the file are arguably good upstreaming candidates).
[](https://gitpod.io/from-referrer/)
|
large-import
t-data
awaiting-author
|
12/0 |
Mathlib/Data/List/Flatten.lean |
1 |
9 |
['YaelDillies', 'github-actions', 'mathlib4-merge-conflict-bot', 'urkud', 'vihdzp'] |
nobody |
6-61008 6 days ago |
6-61008 6 days ago |
3-56140 3 days |
| 31836 |
hanwenzhu author:hanwenzhu |
chore(MeasureTheory/IntervalIntegral): generalize fundamental theorem of calculus to `HasDerivWithinAt` instead of `HasDerivAt` |
This PR generalizes `HasDerivAt` to `HasDerivWithinAt`, and `DifferentiableAt` to `DifferentiableOn`, for the fundamental theorem of calculus for interval integrals.
I found this during trying to state a skeleton of a proof of a higher-dimensional Taylor's theorem. There, the correct assumption is something like `ContDiffOn n f [[a, b]]`, rather than `∀ x ∈ [[a, b]], ContDiffAt 𝕜 n f [[a, b]] x`, which traces back to this issue.
---
[](https://gitpod.io/from-referrer/)
|
t-measure-probability
t-analysis
awaiting-author
|
143/51 |
Mathlib/Analysis/SpecialFunctions/Integrals/Basic.lean,Mathlib/Analysis/SpecialFunctions/NonIntegrable.lean,Mathlib/MeasureTheory/Constructions/BorelSpace/Order.lean,Mathlib/MeasureTheory/Integral/IntervalIntegral/FundThmCalculus.lean,Mathlib/MeasureTheory/Integral/IntervalIntegral/IntegrationByParts.lean,Mathlib/NumberTheory/AbelSummation.lean,Mathlib/NumberTheory/LSeries/SumCoeff.lean |
7 |
9 |
['github-actions', 'hanwenzhu', 'sgouezel'] |
sgouezel assignee:sgouezel |
6-48231 6 days ago |
7-72350 7 days ago |
6-17373 6 days |
| 30998 |
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/)
---
*This PR continues the work from #24350.*
*Original PR: https://github.com/leanprover-community/mathlib4/pull/24350* |
t-algebra label:t-algebra$ |
339/0 |
Mathlib.lean,Mathlib/FieldTheory/Perfect.lean,Mathlib/FieldTheory/SeparablyGenerated.lean,Mathlib/RingTheory/AlgebraicIndependent/Defs.lean |
4 |
25 |
['alreadydone', 'erdOne', 'github-actions', 'grunweg', 'jcommelin', 'kckennylau', 'leanprover-bot', 'leanprover-radar', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
joelriou assignee:joelriou |
6-41607 6 days ago |
10-24879 10 days ago |
22-32212 22 days |
| 32126 |
nielsvoss author:nielsvoss |
feat(Analysis/Normed/Operator): definition of singular values for linear maps |
This PR defines a generalization of singular values, the approximation numbers, for continuous linear maps between normed vector spaces. It proves basic lemmas about the approximation numbers and shows that for finite-dimensional vector spaces, the approximation numbers coincide with the standard definition of singular values.
See the discussion on Zulip: https://leanprover.zulipchat.com/#narrow/channel/217875-Is-there-code-for-X.3F/topic/Singular.20Value.20Decomposition/with/558914024
Co-authored-by: Arnav Mehta
Co-authored-by: Rawad Kansoh
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-analysis
WIP
|
331/0 |
Mathlib/Analysis/Normed/Operator/SingularValues.lean |
1 |
2 |
['github-actions', 'nielsvoss'] |
nobody |
6-39729 6 days ago |
9-4596 9 days ago |
0-0 0 seconds |
| 31754 |
dagurtomas author:dagurtomas |
feat: light profinite sets are injective objects |
---
[](https://gitpod.io/from-referrer/)
|
t-condensed
t-topology
t-category-theory
WIP
|
385/0 |
Mathlib.lean,Mathlib/Topology/Category/LightProfinite/Injective.lean,Mathlib/Topology/Separation/Profinite.lean |
3 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
6-35290 6 days ago |
15-61009 15 days ago |
0-2 2 seconds |
| 31987 |
saodimao20 author:saodimao20 |
feat: add monotonicity and relation lemmas for mgf and cgf |
Add two lemmas about moment-generating and cumulant-generating functions:
- `mgf_mono_in_t_of_nonneg`: For nonnegative random variables, the mgf is monotone in the parameter `t`
- `cgf_zero_of_mgf_one`: The cgf equals zero iff the mgf equals one
These lemmas are useful for studying properties of mgf and cgf in probability theory.
Contributed by sequential-intelligence-lab(SIL), University of Virginia
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-measure-probability
|
21/0 |
Mathlib/Probability/Moments/Basic.lean |
1 |
5 |
['DavidLedvinka', 'github-actions'] |
RemyDegenne assignee:RemyDegenne |
6-32609 6 days ago |
12-5480 12 days ago |
12-5520 12 days |
| 31838 |
qawbecrdtey author:qawbecrdtey |
chore(Data/Finset/Basic): use more dot notation in `Data.Finset.Basic` |
---
- [x] depends on: #31837
[](https://gitpod.io/from-referrer/)
|
t-data |
37/37 |
Mathlib/Data/Finset/Basic.lean |
1 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
TwoFX assignee:TwoFX |
6-26034 6 days ago |
10-23467 10 days ago |
10-48565 10 days |
| 32004 |
jsm28 author:jsm28 |
feat(Geometry/Euclidean/Angle/Sphere): unoriented law of sines with circumradius |
We have the law of sines involving the circumradius for oriented angles in `Mathlib.Geometry.Euclidean.Angle.Sphere`, and for unoriented angles in a form not involving the circumradius in `Mathlib.Geometry.Euclidean.Triangle`. Add a version involving the circumradius but with unoriented angles, deduced from the oriented angles version via moving to a two-dimensional subspace and picking an orientation.
---
- [ ] depends on: #32001
- [ ] depends on: #32002
[](https://gitpod.io/from-referrer/)
|
t-euclidean-geometry |
36/1 |
Mathlib/Geometry/Euclidean/Angle/Sphere.lean |
1 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
JovanGerb assignee:JovanGerb |
6-26033 6 days ago |
10-46456 10 days ago |
10-47248 10 days |
| 32019 |
jsm28 author:jsm28 |
feat(Geometry/Euclidean/Projection): `map` and subtype lemmas |
Add lemmas about mapping `orthogonalProjection`, `reflection` and `orthogonalProjectionSpan` under an affine isometry, and in particular mapping from a subspace to the full space.
---
- [x] depends on: #32016
[](https://gitpod.io/from-referrer/)
|
t-euclidean-geometry |
55/0 |
Mathlib/Geometry/Euclidean/Projection.lean |
1 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
JovanGerb assignee:JovanGerb |
6-26032 6 days ago |
10-55552 10 days ago |
10-56367 10 days |
| 30757 |
SnirBroshi author:SnirBroshi |
feat(Combinatorics/SimpleGraph/Acyclic): `singletonGraph` and `subgraphOfAdj` are trees |
---
[](https://gitpod.io/from-referrer/)
|
t-combinatorics |
26/1 |
Mathlib/Combinatorics/SimpleGraph/Acyclic.lean,Mathlib/Combinatorics/SimpleGraph/Subgraph.lean |
2 |
3 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
kmill assignee:kmill |
6-21163 6 days ago |
6-21189 6 days ago |
39-47854 39 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 |
5-84012 5 days ago |
163-18527 5 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$ |
439/0 |
Mathlib/Topology/Algebra/Krasner.lean |
1 |
n/a |
['github-actions', 'jjdishere', 'mathlib4-merge-conflict-bot'] |
nobody |
5-83974 5 days ago |
unknown |
unknown |
| 30736 |
alreadydone author:alreadydone |
feat(RingTheory): Picard group of a domain is isomorphic to ClassGroup |
---
- [x] depends on: #30657
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebra
label:t-algebra$ |
389/88 |
Mathlib/Algebra/Algebra/Bilinear.lean,Mathlib/Algebra/Algebra/Operations.lean,Mathlib/Data/Set/Semiring.lean,Mathlib/LinearAlgebra/Span/Defs.lean,Mathlib/RingTheory/ClassGroup.lean,Mathlib/RingTheory/FractionalIdeal/Basic.lean,Mathlib/RingTheory/FractionalIdeal/Operations.lean,Mathlib/RingTheory/Localization/Defs.lean,Mathlib/RingTheory/PicardGroup.lean,docs/references.bib |
10 |
15 |
['alreadydone', 'erdOne', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
mariainesdff assignee:mariainesdff |
5-79776 5 days ago |
5-79784 5 days ago |
14-66172 14 days |
| 32232 |
grunweg author:grunweg |
chore: tidy flexible linter exceptions |
- Remove a now-obsolete comment from Mathlib.Init.
- Remove a few now-superfluous exceptions. (A fair number of them were fixed during review, but the exception removal did not get merged.)
- Tweak some annotation comments: move some on the same line, to make it easier to audit the remaining cases (and their reasons) via searching.
---
[](https://gitpod.io/from-referrer/)
|
|
9/30 |
Mathlib/Algebra/Polynomial/Bivariate.lean,Mathlib/Analysis/AbsoluteValue/Equivalence.lean,Mathlib/Analysis/Complex/Exponential.lean,Mathlib/Analysis/SpecialFunctions/ContinuousFunctionalCalculus/PosPart/Basic.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Complex.lean,Mathlib/CategoryTheory/Bicategory/Adjunction/Mate.lean,Mathlib/CategoryTheory/Comma/Over/Pullback.lean,Mathlib/CategoryTheory/Limits/Constructions/Equalizers.lean,Mathlib/CategoryTheory/Limits/Shapes/Products.lean,Mathlib/CategoryTheory/Products/Basic.lean,Mathlib/Combinatorics/Additive/FreimanHom.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/Init.lean |
13 |
1 |
['github-actions'] |
nobody |
5-66317 5 days ago |
5-78526 5 days ago |
5-78503 5 days |
| 31733 |
jsm28 author:jsm28 |
feat(Geometry/Euclidean/Incenter): `orthRadius` lemmas |
Add lemmas, in the case where the dimensions are such that the simplex spans the whole space, exspheres are not merely tangent to the faces but the faces are the full tangent spaces (`orthRadius`).
---
- [x] depends on: #31727
- [x] depends on: #31728
- [x] depends on: #31731
[](https://gitpod.io/from-referrer/)
|
t-euclidean-geometry |
29/0 |
Mathlib/Geometry/Euclidean/Incenter.lean |
1 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
JovanGerb assignee:JovanGerb |
5-62027 5 days ago |
14-66392 14 days ago |
14-67231 14 days |
| 31780 |
euprunin author:euprunin |
feat: add `grind` annotations for `SimpleGraph.Walk.length_{support,darts,edges}` |
---
Note that the lemma being annotated is
1. already actively used with `grind` via explicit `grind [lemma]` invocations in Mathlib, and
2. already tagged with `@[simp]`.
---
[](https://gitpod.io/from-referrer/)
|
t-combinatorics |
4/4 |
Mathlib/Combinatorics/SimpleGraph/Hamiltonian.lean,Mathlib/Combinatorics/SimpleGraph/Walks/Basic.lean |
2 |
8 |
['SnirBroshi', 'euprunin', 'github-actions', 'leanprover-bot', 'leanprover-radar', 'mathlib4-merge-conflict-bot'] |
awainverse assignee:awainverse |
5-59917 5 days ago |
9-46958 9 days ago |
16-22432 16 days |
| 31092 |
FlAmmmmING author:FlAmmmmING |
feat(Algebra/Group/ForwardDiff.lean): Add theorem `sum_shift_eq_fwdDiff_iter`. |
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-algebra
awaiting-author
label:t-algebra$ |
21/1 |
Mathlib/Algebra/Group/ForwardDiff.lean |
1 |
12 |
['FlAmmmmING', 'Ruben-VandeVelde', 'dagurtomas', 'github-actions', 'mathlib4-merge-conflict-bot'] |
dagurtomas assignee:dagurtomas |
5-58373 5 days ago |
5-58444 5 days ago |
15-12707 15 days |
| 31921 |
DavidLedvinka author:DavidLedvinka |
feat: FiniteExhaustion |
Creates a structure that contains the data of a non-decreasing sequence of finite sets whose union equals some countable set. This is used in the brownian motion project to transfer a theorem that holds over finite sets to a countable set (with monotone convergence).
The design is modelled on CompactExhaustion (of course it can be seen as precisely a special case but I think taking that approach would be much more convoluted).
I didn't want to give this its own file, but I couldn't put it in `Mathlib.Data.Set.Countable` without creating a `large-import` because I needed the fact that product of finite sets is finite, and couldn't find anywhere else sensible to put it that wouldn't create a `large-import`. Would be happy if someone has a better suggestion. |
brownian
t-data
|
105/0 |
Mathlib.lean,Mathlib/Data/Set/FiniteExhaustion.lean,Mathlib/Data/Set/Lattice.lean |
3 |
13 |
['ADedecker', 'DavidLedvinka', 'YaelDillies', 'github-actions'] |
pechersky assignee:pechersky |
5-57123 5 days ago |
9-42386 9 days ago |
12-29104 12 days |
| 32245 |
erdOne author:erdOne |
feat(RingTheory): the `coassoc_simps` simp set |
Co-authored-by: Yaël Dillies
From Toric
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
toric
|
431/0 |
Mathlib.lean,Mathlib/RingTheory/Coalgebra/CoassocSimps.lean,Mathlib/RingTheory/Coalgebra/SimpAttr.lean |
3 |
1 |
['github-actions'] |
nobody |
5-54541 5 days ago |
5-54541 5 days ago |
0-0 0 seconds |
| 31706 |
Thmoas-Guan author:Thmoas-Guan |
feat(Algebra/ModuleCat): `ModuleCat.uliftFunctor` |
Add `ModuleCat.uliftFunctor`
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
awaiting-author
label:t-algebra$ |
97/0 |
Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Ulift.lean |
2 |
10 |
['dagurtomas', 'erdOne', 'github-actions', 'mathlib4-merge-conflict-bot'] |
mattrobball assignee:mattrobball |
5-52021 5 days ago |
5-52021 5 days ago |
10-49026 10 days |
| 30666 |
erdOne author:erdOne |
feat(NumberTheory): every number field has a ramified prime |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-number-theory
awaiting-author
label:t-algebra$ |
225/30 |
Mathlib.lean,Mathlib/Algebra/Ring/Int/Field.lean,Mathlib/NumberTheory/NumberField/Basic.lean,Mathlib/NumberTheory/NumberField/ClassNumber.lean,Mathlib/NumberTheory/NumberField/Cyclotomic/Ideal.lean,Mathlib/NumberTheory/NumberField/Discriminant/Different.lean,Mathlib/NumberTheory/NumberField/ExistsRamified.lean,Mathlib/NumberTheory/RamificationInertia/Basic.lean,Mathlib/RingTheory/Ideal/Norm/AbsNorm.lean,Mathlib/RingTheory/Ideal/Norm/RelNorm.lean,Mathlib/RingTheory/IntegralClosure/IsIntegralClosure/Basic.lean |
11 |
22 |
['erdOne', 'github-actions', 'jcommelin', 'mathlib4-merge-conflict-bot', 'tb65536', 'xroblot'] |
jcommelin assignee:jcommelin |
5-48315 5 days ago |
14-78288 14 days ago |
21-14802 21 days |
| 32118 |
alreadydone author:alreadydone |
feat(Algebra): prerequisites for #31919 |
+ Extract a lemma `exists_aeval_invOf_eq_zero_of_ideal_map_adjoin_add_span_eq_top` that was used in the proof of [stacks#00IB](https://stacks.math.columbia.edu/tag/00IB) and are used to prove both parts of [stacks#090P](https://stacks.math.columbia.edu/tag/090P)
+ Add lemmas on units in a submonoid of a DivisionMonoid/Group(WithZero)
+ Add instances for `integralClosure` and API for integrally closed subrings
+ Add a lemma on `trailingCoeff` of polynomials
+ Fix a statement in `local_hom_TFAE` and rename to `isLocalHom_tfae`
+ Unify the instances `Algebra.ofSubsemiring` and `Algebra.ofSubring`
+ Add `NonUnitalSub(semi)ringClass` instance for `Ideal`
+ Upgrade `ValuationSubring.nonunits` from `Subsemigroup` to `NonUnitalSubring`
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
t-algebra
awaiting-author
label:t-algebra$ |
168/40 |
Mathlib/Algebra/Algebra/Basic.lean,Mathlib/Algebra/Polynomial/Degree/TrailingDegree.lean,Mathlib/NumberTheory/Padics/PadicIntegers.lean,Mathlib/RingTheory/Ideal/Defs.lean,Mathlib/RingTheory/Ideal/Nonunits.lean,Mathlib/RingTheory/IntegralClosure/IntegrallyClosed.lean,Mathlib/RingTheory/LocalRing/LocalSubring.lean,Mathlib/RingTheory/LocalRing/RingHom/Basic.lean,Mathlib/RingTheory/Polynomial/Basic.lean,Mathlib/RingTheory/Polynomial/Ideal.lean,Mathlib/RingTheory/Valuation/AlgebraInstances.lean,Mathlib/RingTheory/Valuation/Integers.lean,Mathlib/RingTheory/Valuation/ValuationSubring.lean |
13 |
26 |
['alreadydone', 'erdOne', 'github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'leanprover-radar'] |
nobody |
5-45904 5 days ago |
5-49940 5 days ago |
3-64404 3 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 `⊤`.
---
- [x] depends on: #28719
- [x] depends on: #28785
[](https://gitpod.io/from-referrer/)
|
t-combinatorics |
30/0 |
Mathlib/Combinatorics/SimpleGraph/Extremal/Turan.lean |
1 |
7 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
b-mehta assignee:b-mehta |
5-26004 5 days ago |
8-72569 8 days ago |
11-70240 11 days |
| 30484 |
vihdzp author:vihdzp |
refactor: override `≤` and `<` in `Function.Injective.semilatticeSup`, etc. |
These constructors now take `LE` and `LT` instance arguments, and proofs that the "induced" relations are equal. This matches the behavior for all other data fields of the same constructors, which avoids diamonds which could otherwise arise.
To recover the old behavior, you can instantiate `LE` and `LT` instances through `PartialOrder.lift` (if they don't exist already), and set the `le` and `lt` fields to `Iff.rfl`.
---
I seem to have (somehow?) changed a syntactic equality on fractional ideals - given that this golfs various proofs and even removes a porting note, I think this change is desirable.
[](https://gitpod.io/from-referrer/)
|
t-order |
394/378 |
Mathlib/Algebra/Lie/Submodule.lean,Mathlib/Algebra/Module/Injective.lean,Mathlib/Algebra/Order/Group/Ideal.lean,Mathlib/Algebra/Order/Kleene.lean,Mathlib/Analysis/Convex/Cone/Dual.lean,Mathlib/Analysis/Normed/Group/Seminorm.lean,Mathlib/Analysis/Seminorm.lean,Mathlib/CategoryTheory/Sites/Precoverage.lean,Mathlib/Combinatorics/Digraph/Basic.lean,Mathlib/Combinatorics/SimpleGraph/Basic.lean,Mathlib/Combinatorics/SimpleGraph/Finsubgraph.lean,Mathlib/Combinatorics/SimpleGraph/Subgraph.lean,Mathlib/Combinatorics/Young/YoungDiagram.lean,Mathlib/FieldTheory/Galois/GaloisClosure.lean,Mathlib/GroupTheory/GroupAction/SubMulAction.lean,Mathlib/MeasureTheory/MeasurableSpace/MeasurablyGenerated.lean,Mathlib/ModelTheory/Definability.lean,Mathlib/NumberTheory/NumberField/FractionalIdeal.lean,Mathlib/Order/BooleanAlgebra/Basic.lean,Mathlib/Order/BooleanSubalgebra.lean,Mathlib/Order/CompleteBooleanAlgebra.lean,Mathlib/Order/CompleteLattice/Basic.lean,Mathlib/Order/CompleteLattice/Lemmas.lean,Mathlib/Order/CompleteSublattice.lean,Mathlib/Order/Concept.lean,Mathlib/Order/Disjoint.lean,Mathlib/Order/Heyting/Basic.lean,Mathlib/Order/Heyting/Regular.lean,Mathlib/Order/Hom/Bounded.lean,Mathlib/Order/Hom/BoundedLattice.lean,Mathlib/Order/Hom/Lattice.lean,Mathlib/Order/Interval/Basic.lean,Mathlib/Order/Lattice.lean,Mathlib/Order/Nucleus.lean,Mathlib/Order/Sublattice.lean,Mathlib/Order/UpperLower/CompleteLattice.lean,Mathlib/RingTheory/DedekindDomain/Different.lean,Mathlib/RingTheory/DedekindDomain/Factorization.lean,Mathlib/RingTheory/DedekindDomain/Ideal/Basic.lean,Mathlib/RingTheory/DividedPowers/SubDPIdeal.lean,Mathlib/RingTheory/Filtration.lean,Mathlib/RingTheory/FractionalIdeal/Basic.lean,Mathlib/RingTheory/FractionalIdeal/Extended.lean,Mathlib/RingTheory/FractionalIdeal/Inverse.lean,Mathlib/RingTheory/FractionalIdeal/Operations.lean,Mathlib/RingTheory/GradedAlgebra/Homogeneous/Ideal.lean,Mathlib/Topology/Algebra/Group/ClosedSubgroup.lean,Mathlib/Topology/Algebra/Group/GroupTopology.lean,Mathlib/Topology/Algebra/Module/ClosedSubmodule.lean,Mathlib/Topology/Algebra/OpenSubgroup.lean,Mathlib/Topology/ContinuousMap/Bounded/Normed.lean,Mathlib/Topology/ContinuousMap/CompactlySupported.lean,Mathlib/Topology/ContinuousMap/Ordered.lean,Mathlib/Topology/DiscreteQuotient.lean,Mathlib/Topology/Sets/Closeds.lean,Mathlib/Topology/Sets/Compacts.lean,Mathlib/Topology/Sets/Opens.lean,Mathlib/Topology/Sets/Order.lean |
58 |
38 |
['Vierkantor', 'YaelDillies', 'github-actions', 'leanprover-bot', 'leanprover-radar', 'mathlib4-merge-conflict-bot', 'plp127', 'vihdzp'] |
bryangingechen assignee:bryangingechen |
5-26003 5 days ago |
8-48434 8 days ago |
14-33120 14 days |
| 30921 |
EtienneC30 author:EtienneC30 |
feat: characterizing Gaussian measures through the shape of the characteristic function |
Prove that Gaussian measures over a Banach space `E` are exactly those measures `μ` such that there exist `m : E` and `f : StrongDual ℝ E →L[ℝ] StrongDual ℝ E →L[ℝ] ℝ` satisfying `f.toBilinForm.IsPosSemidef` and `charFunDual μ L = exp (L m * I - f L L / 2)`.
Prove that such `m` and `f` are unique and equal to `∫ x, x ∂μ` and `covarianceBilinDual μ`.
Specialize these statements in the case of Hilbert spaces, with `f : E →L[ℝ] E →L[ℝ] ℝ`, `charFun μ t = exp (⟪t, m⟫ * I - f t t / 2)` and `f = covarianceBilin μ`.
---
- [x] depends on: #30371
- [x] depends on: #31564
- [x] depends on: #31566
- [x] depends on: #31567
from BrownianMotion
[](https://gitpod.io/from-referrer/)
|
brownian
t-measure-probability
|
206/0 |
Mathlib.lean,Mathlib/Probability/Distributions/Gaussian/CharFun.lean,Mathlib/Probability/Moments/CovarianceBilinDual.lean |
3 |
4 |
['RemyDegenne', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
kex-y assignee:kex-y |
5-26002 5 days ago |
8-73615 8 days ago |
9-11711 9 days |
| 31141 |
peabrainiac author:peabrainiac |
feat(Analysis/Calculus): parametric integrals over smooth functions are smooth |
Show that for any smooth function `f : H × ℝ → E`, the parametric integral `fun x ↦ ∫ t in a..b, f (x, t) ∂μ` is smooth too.
The argument proceeds inductively, using the fact that derivatives of parametric integrals can themselves be computed as parametric integrals. The necessary lemmas on derivatives of parametric integrals already existed, but took some work to apply due to their generality; we state some convenient special cases.
---
- [x] depends on: #31077
[](https://gitpod.io/from-referrer/)
|
t-analysis |
199/5 |
Mathlib/Analysis/Calculus/ParametricIntegral.lean,Mathlib/Analysis/Calculus/ParametricIntervalIntegral.lean,Mathlib/MeasureTheory/Integral/DominatedConvergence.lean |
3 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
sgouezel assignee:sgouezel |
5-26001 5 days ago |
8-42709 8 days ago |
8-45471 8 days |
| 31180 |
CoolRmal author:CoolRmal |
feat(Analysis): a closed convex set is the intersection of countably many half-spaces in a separable Banach space |
This lemma is needed in the proof of conditional Jensen's inequality: #27953
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-analysis
awaiting-author
|
69/12 |
Mathlib/Analysis/LocallyConvex/Separation.lean,Mathlib/Topology/Compactness/Lindelof.lean |
2 |
40 |
['ADedecker', 'CoolRmal', 'EtienneC30', 'github-actions', 'j-loreaux', 'mathlib4-merge-conflict-bot'] |
nobody |
5-19569 5 days ago |
6-68601 6 days ago |
3-22471 3 days |
| 32267 |
vlad902 author:vlad902 |
feat(SimpleGraph): add `SimpleGraph.HomClass` |
Inspired by [this PR review feedback.](https://github.com/leanprover-community/mathlib4/pull/30129#discussion_r2530032044)
---
[](https://gitpod.io/from-referrer/)
|
t-combinatorics |
4/0 |
Mathlib/Combinatorics/SimpleGraph/Maps.lean |
1 |
1 |
['YaelDillies', 'github-actions'] |
nobody |
4-75540 4 days ago |
4-77471 4 days ago |
4-77507 4 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 |
16 |
['Vierkantor', 'YaelDillies', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-merge-conflict-bot', 'urkud'] |
Vierkantor assignee:Vierkantor |
4-71504 4 days ago |
15-75075 15 days ago |
0-17 17 seconds |
| 32134 |
mitchell-horner author:mitchell-horner |
feat(Topology/Real): theorems linking `IsGLB` with `BddBelow`, `Antitone`, `Tendsto _ atTop` |
Implement theorems linking `IsGLB` (`IsLUB`) with `BddBelow` (`BddAbove`), `Antitone` (`Monotone`), `Tendsto _ atTop`
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-topology
awaiting-author
|
92/8 |
Mathlib/Algebra/Order/Monoid/Canonical/Basic.lean,Mathlib/Topology/Instances/NNReal/Lemmas.lean |
2 |
9 |
['YaelDillies', 'github-actions', 'mitchell-horner'] |
nobody |
4-70476 4 days ago |
4-70476 4 days ago |
0-7314 2 hours |
| 31444 |
harahu author:harahu |
doc(Probability/Martingale/BorelCantelli): polish docstrings |
Fix some typos and inconsistencies in `BorelCantelli`. The issues were found and fixed using Codex.
The most substantive change is going from
$$f_n := \sum_{k < n} \mathbf{1}_{s_{n + 1}} - \mathbb{P}[s_{n + 1} \mid \mathcal{F}_n]$$
to
$$f_n := \sum_{k < n} \big(\mathbf{1}_{s_{k + 1}} - \mathbb{P}[s_{k + 1} \mid \mathcal{F}_k]\big).$$
As far as I can tell, this is more faithful to the contents of the file.
---
[](https://gitpod.io/from-referrer/)
|
t-measure-probability
delegated
|
5/5 |
Mathlib/Probability/Martingale/BorelCantelli.lean |
1 |
4 |
['github-actions', 'grunweg', 'harahu', 'mathlib-bors'] |
nobody |
4-62840 4 days ago |
24-64780 24 days ago |
0-71658 19 hours |
| 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
t-meta
|
67/8 |
Mathlib/MeasureTheory/Integral/Bochner/L1.lean,Mathlib/MeasureTheory/Measure/Decomposition/IntegralRNDeriv.lean,Mathlib/MeasureTheory/Measure/MeasureSpaceDef.lean,Mathlib/MeasureTheory/OuterMeasure/AE.lean,Mathlib/MeasureTheory/OuterMeasure/BorelCantelli.lean,Mathlib/Probability/Notation.lean |
6 |
34 |
['YaelDillies', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'thorimur', 'urkud'] |
RemyDegenne and thorimur assignee:RemyDegenne assignee:thorimur |
4-59274 4 days ago |
29-59521 29 days ago |
29-59479 29 days |
| 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 set, 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.
---
- [x] depends on: #28346
- [x] depends on: #28336
- [x] depends on: #28332
- [x] depends on: #28330
- [x] depends on: #28224
- [x] depends on: #27968
- [x] depends on: #28034
- [x] depends on: #26076
[](https://gitpod.io/from-referrer/)
|
t-algebraic-topology |
107/0 |
Mathlib.lean,Mathlib/AlgebraicTopology/SimplexCategory/Basic.lean,Mathlib/AlgebraicTopology/SimplicialSet/AnodyneExtensions/Pairing.lean,Mathlib/AlgebraicTopology/SimplicialSet/AnodyneExtensions/RankNat.lean |
4 |
n/a |
['github-actions', 'joelriou', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
4-56349 4 days ago |
unknown |
unknown |
| 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
|
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 |
4-51466 4 days ago |
121-81590 3 months ago |
0-1757 29 minutes |
| 30851 |
FormulaRabbit81 author:FormulaRabbit81 |
feat(Topology): prove there exists an embedding of separable metric spaces in the hilbert cube |
---
[](https://gitpod.io/from-referrer/)
- [x] depends on: #30849 |
t-topology |
73/10 |
Mathlib/Topology/Compactness/HilbertCubeEmbedding.lean,Mathlib/Topology/MetricSpace/HausdorffAlexandroff.lean,Mathlib/Topology/MetricSpace/PiNat.lean |
3 |
9 |
['FormulaRabbit81', 'erdOne', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
ADedecker assignee:ADedecker |
4-33596 4 days ago |
4-33596 4 days ago |
24-41650 24 days |
| 28853 |
grunweg author:grunweg |
feat: product of immersions is an immersion |
---
- [x] depends on: #28793
- [x] depends on: #30356 (for simplicity)
- [x] depends on: #28840
[](https://gitpod.io/from-referrer/)
|
t-differential-geometry
awaiting-author
|
161/30 |
Mathlib/Data/Set/Prod.lean,Mathlib/Geometry/Manifold/Immersion.lean,Mathlib/Geometry/Manifold/IsManifold/Basic.lean,Mathlib/Geometry/Manifold/IsManifold/ExtChartAt.lean,Mathlib/Geometry/Manifold/LocalSourceTargetProperty.lean,Mathlib/Topology/OpenPartialHomeomorph.lean |
6 |
14 |
['chrisflav', 'github-actions', 'grunweg', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
4-30358 4 days ago |
4-61296 4 days ago |
0-22179 6 hours |
| 31988 |
winstonyin author:winstonyin |
feat: Uniqueness of implicit function |
As part of the implicit function theorem, the implicit function is locally unique.
I add some lemmas to facilitate the shuffling of factors of Cartesian products in Filter.Eventually statements.
- [ ] depends on: #30595
---
[](https://gitpod.io/from-referrer/)
|
t-analysis |
61/2 |
Mathlib/Analysis/Calculus/Implicit.lean,Mathlib/Analysis/Calculus/ImplicitContDiff.lean,Mathlib/Order/Filter/Prod.lean |
3 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
ADedecker assignee:ADedecker |
4-25995 4 days ago |
7-47563 7 days ago |
7-47550 7 days |
| 32159 |
zhuyizheng author:zhuyizheng |
feat(Order): gaps of disjoint intervals |
Define gaps of a finite set of pairwise disjoint closed intervals.
Part of originally planned #29508
---
[](https://gitpod.io/from-referrer/)
|
new-contributor |
255/0 |
Mathlib.lean,Mathlib/Algebra/BigOperators/Group/Finset/Gaps.lean,Mathlib/Order/Interval/Finset/Gaps.lean |
3 |
2 |
['github-actions'] |
robin-carlier assignee:robin-carlier |
4-25987 4 days ago |
8-26728 8 days ago |
8-26714 8 days |
| 32165 |
yuanyi-350 author:yuanyi-350 |
feat(Real/Trigonometric): Add `sum_cos_arith_progression` and prepare for Dirichlet kernel |
---
[](https://gitpod.io/from-referrer/)
|
t-analysis
awaiting-author
|
68/0 |
Mathlib.lean,Mathlib/Analysis/Fourier/DirichletKernel.lean |
2 |
7 |
['BoltonBailey', 'github-actions', 'urkud', 'yuanyi-350'] |
fpvandoorn assignee:fpvandoorn |
4-19124 4 days ago |
4-19124 4 days ago |
3-82683 3 days |
| 32152 |
Lingyin00 author:Lingyin00 |
feat(GroupTheory/SpecificGroups/Cyclic): generalize the proof of prime_card by not assuming Finite |
previously the proof of prime_card assumes `Finite`, which could derived from the premises of `CommGroup` and `IsSimpleGroup`.
This PR adds a theorem of finiteness of commutative simple group, a theorem of `prime_card` which dosen't assume `Finite`, and a theorem of isomorphism from any commutative simple group to `ZMod p`, where `p` is a prime number.
---
[](https://gitpod.io/from-referrer/)
|
t-group-theory
new-contributor
awaiting-author
|
69/4 |
Mathlib/GroupTheory/SpecificGroups/Cyclic.lean |
1 |
39 |
['Lingyin00', 'github-actions', 'jcommelin', 'plp127', 'tb65536'] |
tb65536 assignee:tb65536 |
4-18835 4 days ago |
4-18835 4 days ago |
3-80717 3 days |
| 32300 |
bjornsolheim author:bjornsolheim |
feat(Geometry/Convex/Cone): define and characterize generating convex cone |
Define the notion of a generating convex cone.
Prove some initial simple lemmas about generating cones.
---
[](https://gitpod.io/from-referrer/)
|
t-convex-geometry
new-contributor
|
18/0 |
Mathlib/Geometry/Convex/Cone/Basic.lean |
1 |
1 |
['github-actions'] |
nobody |
3-79030 3 days ago |
3-79101 3 days ago |
3-79142 3 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
awaiting-author
|
26/5 |
Mathlib/Combinatorics/Enumerative/Partition.lean,Mathlib/Combinatorics/Enumerative/Partition/Basic.lean |
2 |
7 |
['WangYiran01', 'github-actions', 'kckennylau', 'kim-em', 'mathlib4-merge-conflict-bot'] |
b-mehta assignee:b-mehta |
3-75551 3 days ago |
3-75925 3 days ago |
102-52887 102 days |
| 31891 |
jsm28 author:jsm28 |
feat(Geometry/Euclidean/Sphere/OrthRadius): lemmas for setting up and using polars |
Add further lemmas about `orthRadius` that are of use in setting up and using poles and polars. In particular,
`ncard_inter_orthRadius_eq_two_of_dist_lt_radius` is the key part of showing that, in two dimensions, there are exactly two tangents to a circle from a point outside that circle (where the points of tangency lie on the polar of the point from which the two tangents are drawn).
---
Feel free to golf the proof of `ncard_inter_orthRadius_eq_two_of_dist_lt_radius`, it could probably be rather shorter.
---
- [ ] depends on: #32296
[](https://gitpod.io/from-referrer/)
|
t-euclidean-geometry |
88/1 |
Mathlib/Geometry/Euclidean/Sphere/OrthRadius.lean |
1 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
JovanGerb assignee:JovanGerb |
3-71036 3 days ago |
3-72559 3 days ago |
13-30912 13 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
|
57/5 |
Mathlib/RingTheory/PowerSeries/Basic.lean,Mathlib/RingTheory/PowerSeries/Substitution.lean |
2 |
13 |
['Ruben-VandeVelde', 'github-actions', 'mariainesdff', 'mattrobball'] |
mattrobball assignee:mattrobball |
3-69967 3 days ago |
77-74911 2 months ago |
125-8530 125 days |
| 30505 |
mariainesdff author:mariainesdff |
feat(NumberTheory/RatFunc/Ostrowski): prove Ostrowski's theorem for K(X) |
We prove Ostrowski's theorem for the field of rational functions `K(X)`, where `K` is any field.
Co-authored-by: @xgenereux
---
- [x] depends on: #30404
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-number-theory
awaiting-author
label:t-algebra$ |
331/2 |
Mathlib/FieldTheory/RatFunc/AsPolynomial.lean,Mathlib/FieldTheory/RatFunc/Degree.lean,Mathlib/NumberTheory/RatFunc/Ostrowski.lean |
3 |
31 |
['MichaelStollBayreuth', 'alreadydone', 'github-actions', 'mariainesdff', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
MichaelStollBayreuth assignee:MichaelStollBayreuth |
3-69821 3 days ago |
7-62566 7 days ago |
2-41405 2 days |
| 32285 |
awainverse author:awainverse |
chore(ModelTheory/Bundled): Replace CategoryTheory.Bundled |
Replaces the use of CategoryTheory.Bundled L.Structure with a bespoke type for bundled L.Structures,
L.StrucType.
---
[](https://gitpod.io/from-referrer/)
|
t-logic
awaiting-author
|
95/55 |
Mathlib/ModelTheory/Bundled.lean,Mathlib/ModelTheory/Equivalence.lean,Mathlib/ModelTheory/Fraisse.lean,Mathlib/ModelTheory/Order.lean,Mathlib/ModelTheory/Satisfiability.lean |
5 |
2 |
['github-actions', 'jcommelin'] |
nobody |
3-67416 3 days ago |
3-67416 3 days ago |
0-66385 18 hours |
| 31449 |
kim-em author:kim-em |
feat(SemilocallySimplyConnected): definition and alternative formulation |
Note: Proofs in this PR were developed with assistance from Claude. |
awaiting-author |
114/0 |
Mathlib.lean,Mathlib/AlgebraicTopology/FundamentalGroupoid/SemilocallySimplyConnected.lean,Mathlib/Topology/Path.lean |
3 |
3 |
['ADedecker', 'github-actions', 'mathlib4-merge-conflict-bot'] |
ADedecker assignee:ADedecker |
3-66683 3 days ago |
3-66683 3 days ago |
20-82494 20 days |
| 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/)
|
file-removed
t-category-theory
awaiting-author
|
203/64 |
Mathlib.lean,Mathlib/AlgebraicTopology/FundamentalGroupoid/Basic.lean,Mathlib/CategoryTheory/Core.lean,Mathlib/CategoryTheory/Groupoid/FreeGroupoidOfCategory.lean,Mathlib/CategoryTheory/Groupoid/Grpd.lean,Mathlib/CategoryTheory/Groupoid/Grpd/Core.lean,Mathlib/CategoryTheory/Groupoid/Grpd/Free.lean |
7 |
19 |
['Jlh18', 'github-actions', 'joelriou', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
3-63139 3 days ago |
3-63139 3 days ago |
13-59347 13 days |
| 31663 |
xroblot author:xroblot |
feat(Algebra): more instances about `min`, `max`, `iSup` and `iInf` of sub-algebras |
Let `S₁ S₂ : Subalgebra R C`, we add more `Algebra` instances about their min, max, and for `iSup` and `iInf` and the corresponding `IsScalarTower` instances.
We also add the corresponding instances for `IntermediateField F E`. Note that, in this situation, some `IsScalarTower` instances are not added since they can be deduced automatically.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
WIP
label:t-algebra$ |
75/9 |
Mathlib/Algebra/Algebra/Subalgebra/Lattice.lean,Mathlib/FieldTheory/IntermediateField/Adjoin/Defs.lean,Mathlib/RingTheory/LocalProperties/IntegrallyClosed.lean |
3 |
11 |
['github-actions', 'jcommelin', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'leanprover-radar', 'xroblot'] |
mariainesdff assignee:mariainesdff |
3-62656 3 days ago |
3-62656 3 days ago |
15-80365 15 days |
| 31879 |
Thmoas-Guan author:Thmoas-Guan |
feat(Algebra/Homology): Projective dimension in linear equiv |
In this PR, we proved that projective dimension is stable under (semi-) linear equiv of general universe.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
awaiting-author
label:t-algebra$ |
268/0 |
Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/ProjectiveDimension.lean |
2 |
4 |
['Thmoas-Guan', 'dagurtomas', 'github-actions'] |
dagurtomas assignee:dagurtomas |
3-56367 3 days ago |
8-43065 8 days ago |
5-41763 5 days |
| 31746 |
Maldooor author:Maldooor |
refactor(LinearAlgebra/Matrix): generalize positive semidefinite matrices to infinite dimensions |
---
[](https://gitpod.io/from-referrer/)
|
large-import
new-contributor
t-algebra
WIP
label:t-algebra$ |
273/205 |
Mathlib/Data/Finsupp/Defs.lean,Mathlib/Data/Finsupp/Order.lean,Mathlib/Data/Matrix/Diagonal.lean,Mathlib/LinearAlgebra/Matrix/Hermitian.lean,Mathlib/LinearAlgebra/Matrix/PosDef.lean |
5 |
3 |
['Maldooor', 'github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
3-54114 3 days ago |
3-54122 3 days ago |
0-485 8 minutes |
| 32146 |
foderm author:foderm |
feat(ModelTheory): add characterizations of complete theories |
Add `isComplete_eq_complete_theory` and `isComplete_iff_models_elementarily_equivalent` to connect syntactic completeness with semantic properties.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-logic
|
47/0 |
Mathlib/ModelTheory/Satisfiability.lean |
1 |
9 |
['awainverse', 'foderm', 'github-actions'] |
awainverse assignee:awainverse |
3-48009 3 days ago |
8-46734 8 days ago |
8-46778 8 days |
| 31707 |
Thmoas-Guan author:Thmoas-Guan |
feat(Homology): map between `Ext` induced by exact functor |
In this PR, we developed the additive map `Ext(M,N) => Ext(F(M), F(N))` when `F` is exact functor between abelian category. We also developed its linear version when `F` is linear.
Co-authored-by: Wang Jingting
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-category-theory
awaiting-author
label:t-algebra$ |
199/0 |
Mathlib.lean,Mathlib/Algebra/Homology/DerivedCategory/ExactFunctor.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/Map.lean,Mathlib/Algebra/Homology/HomotopyCategory.lean |
4 |
28 |
['Thmoas-Guan', 'erdOne', 'github-actions', 'joelriou', 'mathlib4-merge-conflict-bot'] |
erdOne assignee:erdOne |
3-47311 3 days ago |
3-47311 3 days ago |
7-41631 7 days |
| 32058 |
Thmoas-Guan author:Thmoas-Guan |
feat(Algebra): category version Baer criterion |
In this PR, we added the cateory version of Baer criterion stating that `M` is injective iff `Ext^1(R/I, M)` vanish for all ideal I.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-category-theory
awaiting-author
label:t-algebra$ |
135/0 |
Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Baer.lean |
2 |
3 |
['github-actions', 'joelriou'] |
dagurtomas assignee:dagurtomas |
3-45897 3 days ago |
3-45897 3 days ago |
7-13795 7 days |
| 30920 |
callesonne author:callesonne |
feat(Category/Grpd): define the bicategory of groupoids |
This is a migration of #25561 to a fork.
---
- [x] depends on: #30132
[](https://gitpod.io/from-referrer/)
|
large-import
t-category-theory
|
133/46 |
Mathlib/CategoryTheory/Bicategory/InducedBicategory.lean,Mathlib/CategoryTheory/Category/Grpd.lean,Mathlib/CategoryTheory/ConcreteCategory/Bundled.lean |
3 |
5 |
['Jlh18', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
3-40656 3 days ago |
3-50243 3 days ago |
3-50350 3 days |
| 31121 |
jessealama author:jessealama |
feat: add ComplexShape.EulerCharSigns for generalized Euler characteristic |
Add `ComplexShape.EulerCharSigns` typeclass providing the alternating signs `χ : ι → ℤˣ` for Euler characteristic computations. Instances are provided for `up ℕ`, `down ℕ`, `up ℤ`, and `down ℤ`.
The Euler characteristic definitions (`eulerChar` and `eulerCharTsum`) are defined on `GradedObject` with `ComplexShape` as an explicit parameter. The `HomologicalComplex` versions are abbreviations that apply these to `C.X` and `C.homology`. Both finite and infinite sum versions are provided.
Split from #29713 as suggested by @joelriou. |
t-algebra
t-category-theory
awaiting-author
label:t-algebra$ |
188/0 |
Mathlib.lean,Mathlib/Algebra/Homology/EulerCharacteristic.lean |
2 |
5 |
['github-actions', 'jessealama', 'joelriou', 'mathlib4-merge-conflict-bot'] |
nobody |
3-38492 3 days ago |
14-65549 14 days ago |
12-18361 12 days |
| 32318 |
urkud author:urkud |
feat: `toSpanSingleton` as a continuous linear equivalence |
- Define `ContinuousLinearMap.toSpanSingletonCLE`.
- Use it to golf a proof about `ContDiffOn` and `deriv`.
---
[](https://gitpod.io/from-referrer/)
|
awaiting-zulip
t-topology
|
47/20 |
Mathlib/Analysis/Calculus/ContDiff/Basic.lean,Mathlib/Topology/Algebra/Module/LinearMap.lean,Mathlib/Topology/Algebra/Module/StrongTopology.lean |
3 |
3 |
['github-actions', 'grunweg', 'urkud'] |
nobody |
3-38033 3 days ago |
3-38033 3 days ago |
0-14303 3 hours |
| 31610 |
rudynicolop author:rudynicolop |
feat(Computability/NFA): Kleene star closure for Regular Languages via NFA |
This PR constructs a Kleene star closure for non-epsilon NFAs, and proves that regular languages are closed under Kleene star. The NFA construction is `NFA.kstar`. The main theorems are:
- `NFA.accepts_kstar`: demonstrates that `M.kstar` accepts the Kleene star closure of the language of `M`.
- `IsRegular.kstar`: demonstrates that regular languages are closed under Kleene star.
There is an onging zulip discussion about regular languages in Mathlib: https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Regular.20languages.3A.20the.20review.20queue/with/553759136
This discussion is also tracked at #24205.
Furthermore, the construction and proofs in this PR are heavily inspired by @TpmKranz from his #15651. #15651 supersedes this PR, so if it is accepted then this PR is not needed.
---
- [x] depends on: #31038
[](https://gitpod.io/from-referrer/)
|
t-computability
new-contributor
|
411/1 |
Mathlib/Computability/NFA.lean |
1 |
5 |
['ctchou', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
3-36432 3 days ago |
3-37438 3 days ago |
3-40394 3 days |
| 29624 |
mcdoll author:mcdoll |
feat(LinearAlgebra/LinearPMap): add definition of resolvent and first resolvent identity |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-analysis
awaiting-author
label:t-algebra$ |
179/2 |
Mathlib/LinearAlgebra/LinearPMap.lean |
1 |
9 |
['github-actions', 'j-loreaux', 'mathlib4-merge-conflict-bot', 'mcdoll'] |
kim-em assignee:kim-em |
3-33969 3 days ago |
3-33992 3 days ago |
64-60811 64 days |
| 32195 |
JovanGerb author:JovanGerb |
feat(Data/Finset/Empty): add `@[push]` tags for pushing negation |
This PR tags `Finset.nonempty_iff_ne_empty` and `Finset.not_nonempty_iff_eq_empty` with `@[push]`, so that they can be used in `push_neg`, `by_cases!`, etc.
A bunch of proofs have been golfed using this.
---
[](https://gitpod.io/from-referrer/)
|
|
84/98 |
Mathlib/Algebra/Group/Pointwise/Finset/Basic.lean,Mathlib/Algebra/Module/ZLattice/Basic.lean,Mathlib/Algebra/MonoidAlgebra/Degree.lean,Mathlib/Algebra/Order/Module/HahnEmbedding.lean,Mathlib/Algebra/Polynomial/Basic.lean,Mathlib/Analysis/Convex/SimplicialComplex/Basic.lean,Mathlib/Analysis/LocallyConvex/WithSeminorms.lean,Mathlib/Analysis/SpecialFunctions/Log/PosLog.lean,Mathlib/Combinatorics/Additive/ApproximateSubgroup.lean,Mathlib/Combinatorics/Additive/Energy.lean,Mathlib/Combinatorics/Additive/VerySmallDoubling.lean,Mathlib/Combinatorics/Colex.lean,Mathlib/Combinatorics/Hall/Finite.lean,Mathlib/Combinatorics/SetFamily/AhlswedeZhang.lean,Mathlib/Combinatorics/SetFamily/KruskalKatona.lean,Mathlib/Combinatorics/SimpleGraph/Clique.lean,Mathlib/Data/Finset/BooleanAlgebra.lean,Mathlib/Data/Finset/Card.lean,Mathlib/Data/Finset/Empty.lean,Mathlib/Data/Finset/Filter.lean,Mathlib/Data/Finset/Max.lean,Mathlib/Data/Finset/NAry.lean,Mathlib/Data/Finset/Pi.lean,Mathlib/Data/Finset/Powerset.lean,Mathlib/Data/Finset/Prod.lean,Mathlib/Data/Finset/Sigma.lean,Mathlib/Data/Finset/Sym.lean,Mathlib/Data/Finsupp/Defs.lean,Mathlib/Data/Nat/PrimeFin.lean,Mathlib/GroupTheory/CosetCover.lean,Mathlib/LinearAlgebra/Multilinear/Basic.lean,Mathlib/LinearAlgebra/RootSystem/Base.lean,Mathlib/MeasureTheory/SetAlgebra.lean,Mathlib/NumberTheory/Divisors.lean,Mathlib/Order/Interval/Finset/Basic.lean,Mathlib/Order/Partition/Finpartition.lean,Mathlib/RingTheory/HahnSeries/Multiplication.lean,Mathlib/RingTheory/HahnSeries/Summable.lean,Mathlib/Topology/EMetricSpace/PairReduction.lean |
39 |
11 |
['JovanGerb', 'github-actions', 'grunweg', 'mathlib4-merge-conflict-bot'] |
grunweg assignee:grunweg |
3-31078 3 days ago |
3-31081 3 days ago |
3-61136 3 days |
| 31926 |
kim-em author:kim-em |
experiment: use `grind` more in #31923 |
- [ ] depends on #31929 |
|
26/24 |
Mathlib/Algebra/BigOperators/Finsupp/Basic.lean,Mathlib/Algebra/Polynomial/Reverse.lean,Mathlib/Analysis/Fourier/BoundedContinuousFunctionChar.lean,Mathlib/Data/Finsupp/Basic.lean,Mathlib/Data/Finsupp/Defs.lean,Mathlib/Data/Finsupp/Sigma.lean,Mathlib/Data/Finsupp/Single.lean,Mathlib/Data/List/ToFinsupp.lean,Mathlib/Data/Set/Sigma.lean,Mathlib/Logic/Embedding/Basic.lean |
10 |
3 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
3-30944 3 days ago |
3-30965 3 days ago |
0-0 0 seconds |
| 30826 |
SnirBroshi author:SnirBroshi |
feat(Combinatorics/SimpleGraph/Connectivity/Subgraph): map a walk to its own subgraph |
While this is not very interesting on its own, it opens the possibility of mapping a walk to any graph, given a graph homomorphism from the walk's subgraph.
---
[](https://gitpod.io/from-referrer/)
|
t-combinatorics |
34/0 |
Mathlib/Combinatorics/SimpleGraph/Connectivity/Subgraph.lean |
1 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
b-mehta assignee:b-mehta |
3-26863 3 days ago |
16-19133 16 days ago |
42-44559 42 days |
| 27100 |
staroperator author:staroperator |
feat(ModelTheory): Presburger definability and semilinear sets |
This PR formalizes the classical result that Presburger definable sets are the same as semilinear sets. As an application of this result, we show that the graph of multiplication is not Presburger definable.
---
- [x] depends on: #26896
- [x] depends on: #27081
- [x] depends on: #27087
- [x] depends on: #27414
- [x] depends on: #32123
---
[](https://gitpod.io/from-referrer/)
|
t-logic |
298/0 |
Mathlib.lean,Mathlib/ModelTheory/Arithmetic/Presburger/Definability.lean,Mathlib/ModelTheory/Arithmetic/Presburger/Semilinear/Defs.lean,docs/references.bib |
4 |
6 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
fpvandoorn assignee:fpvandoorn |
3-26027 3 days ago |
6-61651 6 days ago |
8-62079 8 days |
| 30239 |
luigi-massacci author:luigi-massacci |
feat(Analysis/Distribution/ContDiffMapSupportedIn): Add postcomposition by a CLM as a CLM on D_K^n |
A map `T : F →L[𝕜] F'` induces a map `postcompCLM T : 𝓓^{n}_{K}(E, F) →L[𝕜] 𝓓^{n}_{K}(E, F')`
Co-Authored by: @ADedecker
---
- [x] depends on: #30236
- [x] depends on: #30202
- [x] depends on: #30201
- [x] depends on: #30199
- [x] depends on: #30198
- [x] depends on: #30197
(Note: this PR has changed purpose, the original material was included in previous PRs)
[](https://gitpod.io/from-referrer/)
|
t-analysis |
58/3 |
Mathlib/Analysis/Distribution/ContDiffMapSupportedIn.lean |
1 |
5 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
3-26025 3 days ago |
6-38364 6 days ago |
7-52565 7 days |
| 30926 |
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`.
This is a migration of #14089 to a fork.
---
- [ ] depends on: #30895
[](https://gitpod.io/from-referrer/)
|
t-category-theory |
428/63 |
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 |
10 |
['callesonne', 'edegeltje', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
3-26024 3 days ago |
29-43125 29 days ago |
0-1216 20 minutes |
| 31057 |
jsm28 author:jsm28 |
feat(Geometry/Euclidean/Incenter): `reindex` lemmas |
Add lemmas about all the incenter/excenter-related definitions applied to a reindexed simplex.
---
- [x] depends on: #31054
- [x] depends on: #31055
- [x] depends on: #31056
[](https://gitpod.io/from-referrer/)
|
t-euclidean-geometry |
65/1 |
Mathlib/Geometry/Euclidean/Incenter.lean |
1 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
JovanGerb assignee:JovanGerb |
3-26023 3 days ago |
6-82264 6 days ago |
6-82857 6 days |
| 32043 |
thomaskwaring author:thomaskwaring |
feat(Combinatorics/SimpleGraph/Acyclic): characterise maximal acyclic subgraphs |
We characterise subgraphs `H ≤ G` which are maximal among acyclic subgraphs of `G` as those for which `H.Reachable = G.Reachable`. We also prove that if `G` is acyclic and `x` and `y` are not reachable in `G`, then `G ⊔ fromEdgeSet {s(x,y)}` is acyclic.
---
|
new-contributor
t-combinatorics
|
91/0 |
Mathlib/Combinatorics/SimpleGraph/Acyclic.lean |
1 |
1 |
['github-actions'] |
b-mehta assignee:b-mehta |
3-26019 3 days ago |
10-78874 10 days ago |
10-78913 10 days |
| 32124 |
SnirBroshi author:SnirBroshi |
feat(SimpleGraph/Walks/Operations): expand basic drop/take/reverse API |
---
[](https://gitpod.io/from-referrer/)
|
t-combinatorics |
44/0 |
Mathlib/Combinatorics/SimpleGraph/Walks/Operations.lean |
1 |
1 |
['github-actions'] |
awainverse assignee:awainverse |
3-26017 3 days ago |
9-18327 9 days ago |
9-18372 9 days |
| 32201 |
joelriou author:joelriou |
feat(AlgebraicTopology): dimension of simplicial sets |
For a simplicial set `X` and `d : ℕ`, we introduce a typeclass `X.HasDimensionLT d` saying that the dimension of `X` is `< d`, i.e. all nondegenerate simplices of `X` are of dimension `< d`.
---
[](https://gitpod.io/from-referrer/)
|
t-algebraic-topology |
143/0 |
Mathlib.lean,Mathlib/AlgebraicTopology/SimplicialSet/Dimension.lean,Mathlib/AlgebraicTopology/SimplicialSet/StdSimplex.lean |
3 |
1 |
['github-actions'] |
mattrobball assignee:mattrobball |
3-26014 3 days ago |
7-1190 7 days ago |
7-1168 7 days |
| 32337 |
plp127 author:plp127 |
feat: generalize urysohns lemma |
Generalize some of the theorems in the Urysohn's lemma file.
---
[](https://gitpod.io/from-referrer/)
|
t-topology |
8/6 |
Mathlib/Topology/UrysohnsLemma.lean |
1 |
1 |
['github-actions'] |
nobody |
3-25185 3 days ago |
3-25254 3 days ago |
3-25238 3 days |
| 30618 |
wwylele author:wwylele |
feat(Combinatorics): Glaisher's theorem |
This proves Glaisher's theorem, one of the 1000+ theorems. It is also a generalization of [Euler's partition theorem](https://github.com/leanprover-community/mathlib4/blob/master/Archive/Wiedijk100Theorems/Partition.lean), which can be rewritten as a collorary of this (will be in a different PR)
---
- [ ] depends on: #30599
- [ ] depends on #30567
[](https://gitpod.io/from-referrer/)
|
t-combinatorics |
207/16 |
Archive/Wiedijk100Theorems/Partition.lean,Mathlib.lean,Mathlib/Combinatorics/Enumerative/Partition/Basic.lean,Mathlib/Combinatorics/Enumerative/Partition/GenFun.lean,Mathlib/Combinatorics/Enumerative/Partition/Glaisher.lean,Mathlib/RingTheory/PowerSeries/PiTopology.lean,docs/1000.yaml |
7 |
34 |
['AntoineChambert-Loir', 'b-mehta', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'wwylele'] |
b-mehta assignee:b-mehta |
3-23685 3 days ago |
15-64849 15 days ago |
25-43613 25 days |
| 30144 |
alreadydone author:alreadydone |
feat(Data/Nat): kernel reducible binaryRec |
+ Redefine `Nat.binaryRec` to allow kernel reduction.
+ Move some lemmas from Data/Nat/Bitwise to Data/Nat/BinaryRec.
+ Use `nsmulBinRec` for nsmul/zsmul on elliptic curves.
---
[](https://gitpod.io/from-referrer/)
|
t-data
t-algebra
label:t-algebra$ |
95/40 |
Mathlib/Algebra/Group/Defs.lean,Mathlib/Algebra/Group/Prod.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Affine/Point.lean,Mathlib/Data/Nat/BinaryRec.lean,Mathlib/Data/Nat/BitIndices.lean,Mathlib/Data/Nat/Bitwise.lean,Mathlib/Data/Nat/Digits/Defs.lean |
7 |
11 |
['alreadydone', 'astrainfinita', 'github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'mathlib4-merge-conflict-bot'] |
pechersky assignee:pechersky |
3-15899 3 days ago |
7-74066 7 days ago |
53-15644 53 days |
| 29960 |
yonggyuchoimath author:yonggyuchoimath |
feat(Algebra/Category/Ring): equalizers of pushout maps of tensor product inclusions |
This PR defines a ring map `S →ₗ[R] S ⊗[R] S : s ↦ (s ⊗ₜ[R] 1) - (1 ⊗ₜ[R] s)` for an `R`-algebra `S`, and show that its kernel is exactly (the image of) `R` if `S` is faithfully flat over `R`.
Changes:
* `TensorProduct.AlgebraTensorModule.distribBaseChange`: Origianlly takes `M` and `N`, where `M` is an `R`-module with an additional instance `IsScalarTower R A M`. This is unnecessary, so I changed the `M` and `N` into `N` and `Q`, now both of which are merely modules over `R`.
Main results :
* Add compatibility of `Algebra.TensorProduct.includeLeft` (or `Algebra.TensorProduct.includeRight`) with `TensorProduct.AlgebraTensorModule.distribBaseChange` and `LinearMap.lTensor`
* Define `Algebra.TensorProduct.includeLeftSubRight`, which is the `R`-linear map `S →ₗ[R] S ⊗[R] S` sending `s : S` to `(s ⊗ₜ[R] 1) - (1 ⊗ₜ[R] s)`.
* `Algebra.TensorProduct.exactIncludeLeftSubRight_of_faithfullyFlat`: the pair `algebraMap : R → S` and `includeLeftSubRight R S : S → S ⊗[R] S` is exact if `S` is a faithfully flat `R`-algebra.
---
- [x] depends on: #30806 |
new-contributor |
227/1 |
Mathlib.lean,Mathlib/LinearAlgebra/TensorProduct/Tower.lean,Mathlib/RingTheory/TensorProduct/IncludeLeftSubRight.lean,Mathlib/RingTheory/TensorProduct/Maps.lean |
4 |
8 |
['erdOne', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'yonggyuchoimath'] |
nobody |
3-12432 3 days ago |
3-14106 3 days ago |
53-14039 53 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. |
large-import
t-combinatorics
|
53/6 |
Mathlib/Combinatorics/SimpleGraph/Connectivity/WalkDecomp.lean,Mathlib/Combinatorics/SimpleGraph/Walks/Operations.lean,Mathlib/Combinatorics/SimpleGraph/Walks/Subwalks.lean |
3 |
4 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
awainverse assignee:awainverse |
3-6354 3 days ago |
3-6373 3 days ago |
68-67445 68 days |
| 30872 |
rudynicolop author:rudynicolop |
feat(Computability/NFA): NFA closure under concatenation |
This PR proves that regular languages are closed under concatenation via a direct construction on `NFA`s without `εNFA` nor ε-transitions. The main new definitions and results include:
- `M1.concat M2`, the concatenation of `NFA`s `M1` and `M2`, also notated as `M1 * M2`, a direct construction without ε-transitions.
- Theorem `concat_accepts : (M1 * M2).accepts = M1.accepts * M2.accepts`, showing the correctness of the construction.
- Theorem `IsRegular.concat`, showing that regular languages are closed under concatenation.
---
- [x] depends on: #31038
[](https://gitpod.io/from-referrer/)
|
t-computability
new-contributor
awaiting-author
|
150/0 |
Mathlib/Computability/NFA.lean |
1 |
31 |
['YaelDillies', 'ctchou', 'github-actions', 'lambda-fairy', 'mathlib4-dependent-issues-bot', 'rudynicolop'] |
YaelDillies assignee:YaelDillies |
3-5817 3 days ago |
3-84515 3 days ago |
8-68526 8 days |
| 31019 |
vihdzp author:vihdzp |
feat: colex order on finsupps |
---
- [ ] depends on: #30482
[](https://gitpod.io/from-referrer/)
|
|
155/14 |
Mathlib/Data/DFinsupp/Lex.lean,Mathlib/Data/Finsupp/Lex.lean,Mathlib/Order/Synonym.lean |
3 |
4 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
3-5426 3 days ago |
3-5428 3 days ago |
3-5975 3 days |
| 31205 |
jsm28 author:jsm28 |
feat(Analysis/Convex/Side): affine combinations and sides of faces of a simplex |
Add lemmas saying when (in terms of the weights in the combinations) two affine combinations of the vertices of a simplex lie (strictly or weakly) on the same or opposite sides of a face of that simplex opposite a vertex.
---
- [x] depends on: #31204
- [x] depends on: #32150
- [x] depends on: #32161
- [x] depends on: #32164
[](https://gitpod.io/from-referrer/)
|
t-convex-geometry |
161/0 |
Mathlib/Analysis/Convex/Side.lean |
1 |
7 |
['github-actions', 'jcommelin', 'jsm28', 'mathlib4-dependent-issues-bot'] |
YaelDillies assignee:YaelDillies |
3-1199 3 days ago |
7-83434 7 days ago |
17-72890 17 days |
| 32345 |
joelriou author:joelriou |
feat(AlgebraicTopology): relative morphisms of simplicial sets |
Given two simplicial sets `X` and `Y`, and subcomplexes `A` of `X`, and `B` of `Y`, we introduce a type `RelativeMorphism A B φ` of morphisms `X ⟶ Y` which induce a given morphism of simplicial sets `A ⟶ B`. We define homotopies between these relative morphisms and introduce the quotient type of homotopy classes.
(Homotopy groups of Kan complexes will be defined as a particular case of this construction.)
From https://github.com/joelriou/topcat-model-category
---
[](https://gitpod.io/from-referrer/)
|
t-algebraic-topology |
215/1 |
Mathlib.lean,Mathlib/AlgebraicTopology/SimplicialSet/Monoidal.lean,Mathlib/AlgebraicTopology/SimplicialSet/RelativeMorphism.lean,Mathlib/AlgebraicTopology/SimplicialSet/Subcomplex.lean |
4 |
1 |
['github-actions'] |
nobody |
2-83603 2 days ago |
2-86376 2 days ago |
2-86354 2 days |
| 32279 |
joelriou author:joelriou |
feat(CategoryTheory): effective epi in the category of functors to types |
In this PR, we show that epimorphisms in `Type` or `C ⥤ Type _` are regular epimorphisms. In particular, they are effective epimorphisms.
(Part of the definitions may be duplicates of the already existing API.)
---
[](https://gitpod.io/from-referrer/)
|
t-category-theory
WIP
|
129/0 |
Mathlib.lean,Mathlib/CategoryTheory/EffectiveEpi/FunctorToTypes.lean,Mathlib/CategoryTheory/Limits/Types/Coequalizers.lean,Mathlib/CategoryTheory/Limits/Types/EffectiveEpi.lean,Mathlib/CategoryTheory/Limits/Types/Pullbacks.lean |
5 |
1 |
['github-actions'] |
nobody |
2-82050 2 days ago |
4-6872 4 days ago |
0-52758 14 hours |
| 31673 |
vasnesterov author:vasnesterov |
chore(Tactic/Order): use `AtomM` |
The `order` tactic uses its own machinery to collect atoms and facts from the context. This PR replaces it with `AtomM` to unify with other tactics like `ring`.
---
- [x] depends on: #26580
[](https://gitpod.io/from-referrer/)
|
t-meta |
175/140 |
Mathlib/Tactic/Order.lean,Mathlib/Tactic/Order/CollectFacts.lean,Mathlib/Tactic/Order/Graph/Basic.lean,Mathlib/Tactic/Order/Graph/Tarjan.lean,Mathlib/Tactic/Order/Preprocessing.lean,Mathlib/Tactic/Order/ToInt.lean,Mathlib/Util/AtomM.lean,MathlibTest/order.lean |
8 |
n/a |
['JovanGerb', 'bryangingechen', 'github-actions', 'grunweg', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'vasnesterov'] |
JovanGerb assignee:JovanGerb |
2-77799 2 days ago |
unknown |
unknown |
| 31812 |
xroblot author:xroblot |
feat(CMField): add `IsCyclotomicExtension.Rat.isCMField` |
We remove the `NumberField` hypothesis in two more results and thus can deduce that any nontrivial cyclotomic extension of `ℚ` is `CM`. In particular, we add the instance:
```lean
instance (K : Type*) [Field K] [CharZero K] [IsCyclotomicExtension ⊤ ℚ K] : IsCMField K
```
---
- [x] depends on: #31811
- [x] depends on: #29688
[](https://gitpod.io/from-referrer/)
|
|
65/19 |
Mathlib/NumberTheory/NumberField/CMField.lean,Mathlib/NumberTheory/NumberField/Cyclotomic/Embeddings.lean,Mathlib/NumberTheory/NumberField/InfinitePlace/Ramification.lean,Mathlib/NumberTheory/NumberField/InfinitePlace/TotallyRealComplex.lean |
4 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
2-77608 2 days ago |
2-77835 2 days ago |
2-80573 2 days |
| 32045 |
xroblot author:xroblot |
chore(Trace/Quotient): move isomorphism to `Localization.AtPrime.Basic` |
This PR move isomorphisms previously defined in `Trace.Quotient` into `Localization.AtPrime.Basic`. The change is purely organizational: `Localization.AtPrime.Basic` is the canonical place for lemmas and constructions about localization at a prime. The isomorphisms are also renamed to match their new namespace:
- `equivQuotMaximalIdealOfIsLocalization` -> `IsLocalization.AtPrime.equivQuotMaximalIdeal`
- `quotMapEquivQuotMapMaximalIdealOfIsLocalization` -> `IsLocalization.AtPrime.equivQuotMapMaximalIdeal`
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory |
142/108 |
Mathlib/RingTheory/Localization/AtPrime/Basic.lean,Mathlib/RingTheory/Trace/Quotient.lean |
2 |
1 |
['github-actions'] |
nobody |
2-75500 2 days ago |
2-77069 2 days ago |
2-77522 2 days |
| 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 |
185/6 |
Mathlib/NumberTheory/SelbergSieve.lean |
1 |
36 |
['FLDutchmann', 'MichaelStollBayreuth', 'bryangingechen', 'github-actions', 'jcommelin', 'mathlib-bors', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
MichaelStollBayreuth assignee:MichaelStollBayreuth |
2-71310 2 days ago |
2-71331 2 days ago |
10-72632 10 days |
| 30885 |
erdOne author:erdOne |
chore(RingTheory): better defeqs for `PrimeSpectrum.preimageOrderIsoTensorResidueField` |
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
large-import
|
120/31 |
Mathlib/RingTheory/Ideal/Prime.lean,Mathlib/RingTheory/LocalRing/ResidueField/Fiber.lean,Mathlib/RingTheory/LocalRing/ResidueField/Ideal.lean |
3 |
9 |
['chrisflav', 'erdOne', 'github-actions', 'mathlib4-merge-conflict-bot'] |
chrisflav assignee:chrisflav |
2-69407 2 days ago |
2-69432 2 days ago |
30-81041 30 days |
| 32355 |
bjornsolheim author:bjornsolheim |
feat(Geometry/Convex/Cone): define and characterize finitely generated and simplicial pointed cones |
Added file Simplicial.lean in which we:
* Define finitely generated and simplicial pointed cones.
* Prove lemmas simplicial_bot and Simplicial.fg.
---
[](https://gitpod.io/from-referrer/)
|
t-convex-geometry
new-contributor
|
80/0 |
Mathlib.lean,Mathlib/Geometry/Convex/Cone/Simplicial.lean |
2 |
1 |
['github-actions'] |
nobody |
2-62537 2 days ago |
2-62544 2 days ago |
2-62584 2 days |
| 32359 |
YuvalFilmus author:YuvalFilmus |
feat(LinearAlgebra/Lagrange): Formula for leading coefficient of a polynomial |
Added `leadingCoeff_interpolate`, which gives a formula for the leading coefficient of a polynomial that follows from Lagrange interpolation.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-algebra
label:t-algebra$ |
50/0 |
Mathlib/LinearAlgebra/Lagrange.lean |
1 |
3 |
['YuvalFilmus', 'github-actions'] |
nobody |
2-58056 2 days ago |
2-58186 2 days ago |
2-58221 2 days |
| 29713 |
jessealama author:jessealama |
feat (Algebra/Homology): add Euler–Poincaré formula |
This PR builds on the generalized Euler characteristic framework from #31121 to prove the Euler-Poincaré formula for chain complexes.
PR #31121 defines the Euler characteristic for general homological complexes. This PR specializes those definitions to ℤ-indexed chain complexes and proves the main Euler-Poincaré theorem.
### Main result (in `EulerPoincare.lean`)
* `ChainComplex.eulerChar_eq_homologyEulerChar`: For ℤ-indexed bounded chain complexes of finite-dimensional modules over a division ring, the alternating sum of chain dimensions equals the alternating sum of homology dimensions.
---
Builds on: #31121
Related to: #29639, #29643, #29646 |
new-contributor
t-algebra
awaiting-author
label:t-algebra$ |
515/0 |
Mathlib.lean,Mathlib/Algebra/Homology/EulerCharacteristic.lean,Mathlib/Algebra/Homology/EulerPoincare.lean |
3 |
24 |
['github-actions', 'jessealama', 'joelriou', 'kim-em', 'mathlib4-merge-conflict-bot'] |
dagurtomas assignee:dagurtomas |
2-57578 2 days ago |
14-65833 14 days ago |
37-64248 37 days |
| 28895 |
yury-harmonic author:yury-harmonic |
feat(NumberTheory): prove Zsigmondy's theorem |
---
- [x] depends on: #28879
- [x] depends on: #28825
- [x] depends on: #28833
- [x] depends on: #28888
- [x] depends on: #28830
- [x] depends on: #28765
- [x] depends on: #28886
- [x] depends on: #28934
[](https://gitpod.io/from-referrer/)
|
|
1307/0 |
Mathlib.lean,Mathlib/NumberTheory/Zsigmondy.lean |
2 |
8 |
['dupuisf', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'yury-harmonic'] |
nobody |
2-55550 2 days ago |
2-55569 2 days ago |
0-0 0 seconds |
| 31845 |
smmercuri author:smmercuri |
feat: `UniformSpace.Completion.mapRingEquiv` |
lifts a ring isomorphism between uniform rings to a ring isomorphism between their uniform space completions
---
[](https://gitpod.io/from-referrer/)
|
t-topology
awaiting-author
|
24/5 |
Mathlib/Topology/Algebra/UniformRing.lean |
1 |
7 |
['ADedecker', 'github-actions', 'j-loreaux', 'smmercuri'] |
j-loreaux assignee:j-loreaux |
2-54108 2 days ago |
2-54108 2 days ago |
4-84128 4 days |
| 31492 |
fcoUnda author:fcoUnda |
Nthroot improvement |
Resolve TODO for nthroot, replacing the dependency on the arithmetic geometric mean inequality by some inequalities on powers of binomials.
---
- [ ] depends on: #31502
[](https://gitpod.io/from-referrer/)
|
awaiting-zulip
new-contributor
t-analysis
|
71/33 |
Mathlib/Analysis/SpecialFunctions/Pow/NthRootLemmas.lean |
1 |
19 |
['fcoUnda', 'github-actions', 'j-loreaux', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'urkud'] |
j-loreaux assignee:j-loreaux |
2-53387 2 days ago |
2-53411 2 days ago |
5-77585 5 days |
| 29942 |
smmercuri author:smmercuri |
feat(InfinitePlace/Completion): embeddings of `w.Completion` factor through embeddings of `v.Completion` when `w` extends `v` |
If `w : v.Extension L` is an extension of `v : InfinitePlace K` to `L`, then `extensionEmbedding w : L →+* ℂ` factors through `extensionEmbedding v : K →+* ℂ`.
---
- [x] depends on: #27978
- [x] depends on: #29969
- [x] depends on: #29944
[](https://gitpod.io/from-referrer/)
|
FLT |
89/14 |
Mathlib/Analysis/Normed/Field/WithAbs.lean,Mathlib/NumberTheory/NumberField/InfinitePlace/Completion.lean,Mathlib/NumberTheory/NumberField/InfinitePlace/Embeddings.lean,Mathlib/NumberTheory/NumberField/InfinitePlace/Ramification.lean,Mathlib/Topology/MetricSpace/Completion.lean |
5 |
5 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
joelriou assignee:joelriou |
2-49810 2 days ago |
6-49780 6 days ago |
6-50877 6 days |
| 32357 |
YuvalFilmus author:YuvalFilmus |
feat(Polynomial/Roots): add a theorem for computing roots |
The theorem `roots_eq_of_degree` shows that S is the set of roots of a degree d polynomial P if #S = d and P(x) = 0 for every x in S.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-algebra
label:t-algebra$ |
14/0 |
Mathlib/Algebra/Polynomial/Roots.lean |
1 |
3 |
['LLaurance', 'github-actions'] |
nobody |
2-48059 2 days ago |
2-58965 2 days ago |
2-59003 2 days |
| 32089 |
erdOne author:erdOne |
feat(Analysis): derivative of Weierstrass ℘ |
---
[](https://gitpod.io/from-referrer/)
|
maintainer-merge
t-analysis
|
300/3 |
Mathlib/Analysis/SpecialFunctions/Elliptic/Weierstrass.lean |
1 |
17 |
['erdOne', 'github-actions', 'j-loreaux', 'loefflerd', 'mathlib4-merge-conflict-bot'] |
nobody |
2-46452 2 days ago |
2-47119 2 days ago |
8-67826 8 days |
| 32360 |
YuvalFilmus author:YuvalFilmus |
feat(Chebyshev): degree, leadingCoeff, eval_neg |
Calculated the degree and leading coefficients of Chebyshev T and U, as well as formulas for T(-x) and U(-x).
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
new-contributor
|
155/2 |
Mathlib/RingTheory/Polynomial/Chebyshev.lean |
1 |
7 |
['LLaurance', 'YuvalFilmus', 'github-actions'] |
nobody |
2-46380 2 days ago |
2-57700 2 days ago |
2-57737 2 days |
| 32365 |
yury-harmonic author:yury-harmonic |
feat: `norm_num` extension for `IsSquare` |
---
[](https://gitpod.io/from-referrer/)
|
t-meta |
189/0 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/NormNum/IsSquare.lean,MathlibTest/norm_num_ext.lean |
4 |
1 |
['github-actions'] |
nobody |
2-43849 2 days ago |
2-47068 2 days ago |
2-47104 2 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 |
2-43725 2 days ago |
121-81574 3 months ago |
28-81831 28 days |
| 32327 |
EtienneC30 author:EtienneC30 |
chore(Probability): split `Independence.Kernel` |
Create a new folder `Kernel` with two files: `Indep` is about independence of families of sets and sigma-algebras, while `IndepFun` contains the definitions and results about independence of random variables.
---
[](https://gitpod.io/from-referrer/)
|
tech debt
t-measure-probability
awaiting-author
|
1586/1538 |
Mathlib.lean,Mathlib/Probability/Independence/Basic.lean,Mathlib/Probability/Independence/Conditional.lean,Mathlib/Probability/Independence/Kernel.lean,Mathlib/Probability/Independence/Kernel/Indep.lean,Mathlib/Probability/Independence/Kernel/IndepFun.lean |
6 |
3 |
['EtienneC30', 'Ruben-VandeVelde', 'github-actions'] |
nobody |
2-43714 2 days ago |
2-79947 2 days ago |
0-51469 14 hours |
| 31925 |
alreadydone author:alreadydone |
feat(Topology): étalé space associated to a predicate on sections |
---
migrated from #22782
[](https://gitpod.io/from-referrer/)
|
t-topology
awaiting-author
|
899/164 |
Mathlib.lean,Mathlib/AlgebraicGeometry/ProjectiveSpectrum/StructureSheaf.lean,Mathlib/Data/Set/Operations.lean,Mathlib/Geometry/Manifold/Sheaf/Smooth.lean,Mathlib/Logic/Equiv/Basic.lean,Mathlib/Topology/EtaleSpace.lean,Mathlib/Topology/IsLocalHomeomorph.lean,Mathlib/Topology/Sheaves/LocalPredicate.lean,Mathlib/Topology/Sheaves/Sheafify.lean,Mathlib/Topology/Sheaves/Stalks.lean |
10 |
12 |
['adamtopaz', 'alreadydone', 'github-actions'] |
adamtopaz assignee:adamtopaz |
2-41403 2 days ago |
8-34807 8 days ago |
4-81911 4 days |
| 32369 |
metakunt author:metakunt |
feat(RingTheory/Coprime/Lemmas): Add Int.isCoprime_gcdA |
Adds Int.isCoprime_gcdA |
t-ring-theory
new-contributor
|
4/0 |
Mathlib/RingTheory/Coprime/Lemmas.lean |
1 |
1 |
['github-actions'] |
nobody |
2-41140 2 days ago |
2-43057 2 days ago |
2-43096 2 days |
| 32188 |
euprunin author:euprunin |
feat: add `grind` annotation for `ENNReal.inv_eq_zero` |
---
Note that the lemma being annotated is
1. already actively used with `grind` via explicit `grind [lemma]` invocations in Mathlib, and
2. already tagged with `@[simp]`.
---
[](https://gitpod.io/from-referrer/)
|
t-data |
4/5 |
Mathlib/Data/ENNReal/Inv.lean |
1 |
5 |
['euprunin', 'github-actions', 'leanprover-bot', 'leanprover-radar', 'metakunt'] |
TwoFX assignee:TwoFX |
2-40924 2 days ago |
7-42380 7 days ago |
7-42415 7 days |
| 32085 |
dagurtomas author:dagurtomas |
feat(CategoryTheory): sheaf categories are regular epi categories |
---
- [x] depends on: #32086
[](https://gitpod.io/from-referrer/)
|
t-category-theory
WIP
|
253/0 |
Mathlib/CategoryTheory/EffectiveEpi/Sheaf.lean,Mathlib/CategoryTheory/Limits/FunctorCategory/Shapes/Pullbacks.lean,Mathlib/CategoryTheory/Limits/Shapes/RegularMono.lean |
3 |
7 |
['dagurtomas', 'github-actions', 'joelriou', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
2-35212 2 days ago |
3-16812 3 days ago |
0-1 1 second |
| 30391 |
rudynicolop author:rudynicolop |
feat(Data/List): list splitting definitions and lemmas |
This PR continues the work from #24395.
Original PR: https://github.com/leanprover-community/mathlib4/pull/24395 |
t-data
new-contributor
|
108/2 |
Mathlib/Data/List/Perm/Lattice.lean,Mathlib/Data/List/TakeDrop.lean |
2 |
36 |
['BoltonBailey', 'github-actions', 'kckennylau', 'mathlib4-merge-conflict-bot', 'rudynicolop'] |
TwoFX assignee:TwoFX |
2-31498 2 days ago |
3-28663 3 days ago |
51-28749 51 days |
| 32375 |
erdOne author:erdOne |
feat(RingTheory): More API for `Ideal.ResidueField` |
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory |
75/21 |
Mathlib/RingTheory/LocalRing/ResidueField/Ideal.lean,Mathlib/RingTheory/LocalRing/ResidueField/Instances.lean,Mathlib/RingTheory/Spectrum/Prime/Polynomial.lean,Mathlib/RingTheory/Spectrum/Prime/RingHom.lean |
4 |
1 |
['github-actions'] |
nobody |
2-30596 2 days ago |
2-30596 2 days ago |
2-30655 2 days |
| 26985 |
agjftucker author:agjftucker |
feat(Analysis/Calculus/Implicit): define implicitFunOfProdDomain |
This PR continues the work from #16743.
Original PR: https://github.com/leanprover-community/mathlib4/pull/16743
---
- [x] depends on: #28352
[](https://gitpod.io/from-referrer/) |
new-contributor
t-analysis
|
108/2 |
Mathlib/Analysis/Calculus/Implicit.lean |
1 |
8 |
['github-actions', 'j-loreaux', 'mathlib-bors', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
hrmacbeth assignee:hrmacbeth |
2-30372 2 days ago |
5-31216 5 days ago |
0-0 0 seconds |
| 32116 |
LessnessRandomness author:LessnessRandomness |
feat(Geometry/Euclidean/Angle/Unoriented/TriangleInequality): Add criterion for equality case |
The PR fills `proof_wanted` in the file `TriangleInequality.lean` (criterion for equality in the triangle inequality for angles).
---
- [ ] depends on: #32100
[](https://gitpod.io/from-referrer/)
|
t-euclidean-geometry |
137/33 |
Mathlib/Geometry/Euclidean/Angle/Unoriented/TriangleInequality.lean |
1 |
25 |
['JovanGerb', 'LessnessRandomness', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'themathqueen'] |
jsm28 assignee:jsm28 |
2-29505 2 days ago |
6-73126 6 days ago |
6-78137 6 days |
| 29393 |
staroperator author:staroperator |
feat(SetTheory/ZFC): `card (V_ o) = preBeth o` |
---
- [x] depends on: #26544
- [x] depends on: #29351
- [x] depends on: #29365
[](https://gitpod.io/from-referrer/)
|
large-import
t-set-theory
|
37/4 |
Mathlib/SetTheory/ZFC/Ordinal.lean,Mathlib/SetTheory/ZFC/VonNeumann.lean |
2 |
5 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'staroperator', 'vihdzp'] |
alreadydone assignee:alreadydone |
2-26013 2 days ago |
6-16092 6 days ago |
6-18718 6 days |
| 31876 |
mcdoll author:mcdoll |
feat(Analysis/Distribution): integration by parts for Schwartz functions |
---
- [x] depends on: #32084
[](https://gitpod.io/from-referrer/)
|
t-analysis |
62/5 |
Mathlib/Analysis/Distribution/SchwartzSpace.lean |
1 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
ADedecker assignee:ADedecker |
2-26009 2 days ago |
2-37843 2 days ago |
2-37821 2 days |
| 31967 |
bwangpj author:bwangpj |
feat: IrreducibleSpace.of_openCover |
Irreducibility can be checked on an open cover with pairwise non-empty intersections.
This contribution was created as part of the Heidelberg Lean workshop "Formalising algebraic geometry" in November 2025.
Co-authored-by: Christian Merten @chrisflav
---
[](https://gitpod.io/from-referrer/)
|
t-topology |
60/0 |
Mathlib/Topology/Irreducible.lean,Mathlib/Topology/Sets/OpenCover.lean,Mathlib/Topology/Sets/Opens.lean |
3 |
12 |
['bwangpj', 'chrisflav', 'erdOne', 'github-actions'] |
alreadydone assignee:alreadydone |
2-26008 2 days ago |
5-60035 5 days ago |
7-62503 7 days |
| 32160 |
SnirBroshi author:SnirBroshi |
feat(Combinatorics/SimpleGraph/Walks): helper theorems about `darts` and `support` |
---
[](https://gitpod.io/from-referrer/)
|
t-combinatorics |
40/0 |
Mathlib/Combinatorics/SimpleGraph/Walks/Basic.lean,Mathlib/Combinatorics/SimpleGraph/Walks/Traversal.lean |
2 |
1 |
['github-actions'] |
kmill assignee:kmill |
2-26006 2 days ago |
8-23640 8 days ago |
8-23675 8 days |
| 32238 |
YaelDillies author:YaelDillies |
feat(Combinatorics/SimpleGraph): distributivity of box product over sum |
From ProofBench
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-combinatorics
|
21/2 |
Mathlib/Combinatorics/SimpleGraph/Prod.lean |
1 |
1 |
['github-actions'] |
kmill assignee:kmill |
2-26003 2 days ago |
5-63350 5 days ago |
5-63386 5 days |
| 32259 |
jsm28 author:jsm28 |
feat(Analysis/SpecialFunctions/Trigonometric/Angle): `toReal` addition lemmas |
Add two lemmas
```lean
lemma toReal_add_eq_toReal_add_toReal {θ ψ : Angle} (hθ : θ ≠ π) (hψ : ψ ≠ π)
(hs : θ.sign ≠ ψ.sign ∨ θ.sign = (θ + ψ).sign) : (θ + ψ).toReal = θ.toReal + ψ.toReal := by
```
```lean
lemma abs_toReal_add_eq_two_pi_sub_abs_toReal_add_abs_toReal {θ ψ : Angle} (hs : θ.sign = ψ.sign)
(hsa : θ.sign ≠ (θ + ψ).sign) : |(θ + ψ).toReal| = 2 * π - (|θ.toReal| + |ψ.toReal|) := by
```
about `(θ + ψ).toReal`. Also add a lemma `abs_toReal_neg` used in proving them, and lemmas `sign_two_nsmul_eq_neg_sign_iff` and `sign_two_zsmul_eq_neg_sign_iff` (analogous to existing `sign_two_nsmul_eq_sign_iff` and `sign_two_zsmul_eq_sign_iff`) that are of use together with the `toReal` lemmas in relating oriented and unoriented angle bisection results.
---
Feel free to golf.
---
[](https://gitpod.io/from-referrer/)
|
t-analysis |
120/0 |
Mathlib/Analysis/SpecialFunctions/Trigonometric/Angle.lean |
1 |
1 |
['github-actions'] |
j-loreaux assignee:j-loreaux |
2-26001 2 days ago |
5-28562 5 days ago |
5-28541 5 days |
| 32372 |
bwangpj author:bwangpj |
feat: InfiniteGalois.normalAutEquivQuotient |
If `H` is a _closed_ normal subgroup of `Gal(K / k)`, then `Gal(fixedField H / k)` is isomorphic to `Gal(K / k) ⧸ H`.
---
[](https://gitpod.io/from-referrer/)
|
|
17/0 |
Mathlib/FieldTheory/Galois/Infinite.lean |
1 |
1 |
['github-actions'] |
nobody |
2-13419 2 days ago |
2-33291 2 days ago |
2-33268 2 days |
| 32371 |
KaiErikNiermann author:KaiErikNiermann |
fix: minor error in comment of example for natural transformation |
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
easy
|
1/1 |
Mathlib/CategoryTheory/NatTrans.lean |
1 |
2 |
['LLaurance', 'github-actions'] |
nobody |
2-2908 2 days ago |
2-3067 2 days ago |
2-37944 2 days |
| 32323 |
LLaurance author:LLaurance |
feat(Combinatorics/SimpleGraph/Connectivity): exists vertex adjacent to any vertex of a nontrivial connected graph |
---
[](https://gitpod.io/from-referrer/)
|
t-combinatorics |
15/0 |
Mathlib/Combinatorics/SimpleGraph/Connectivity/Connected.lean,Mathlib/Combinatorics/SimpleGraph/Connectivity/Subgraph.lean |
2 |
1 |
['github-actions'] |
nobody |
2-1232 2 days ago |
3-50385 3 days ago |
3-53114 3 days |
| 31766 |
SuccessMoses author:SuccessMoses |
feat(Topology/EMetricSpace): continuity of arc length |
fixes #31751
- [x] Topology/EMetricSpace/Arclength.lean
- [ ] Topology/EmetricSpace/PathEMetric.lean
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
awaiting-author
|
442/0 |
Mathlib.lean,Mathlib/Topology/EMetricSpace/Arclength.lean |
2 |
3 |
['SuccessMoses', 'github-actions', 'grunweg'] |
nobody |
2-68 2 days ago |
8-29304 8 days ago |
0-8426 2 hours |
| 31908 |
YaelDillies author:YaelDillies |
feat: Bernoulli random variables |
Define the product distribution of `p`-Bernoulli random variables a measure on `Set ι`.
It is important in applications to be able to restrict the product to a subset `u` of `ι`, eg in #31364 I define the `G(V, p)` distribution of binomial random graphs by setting `ι := Sym2 V` and `u := {e |¬ e.IsDiag}`.
---
- [x] depends on: #31909
- [x] depends on: #31911
- [x] depends on: #32096
- [x] depends on: #32287
[](https://gitpod.io/from-referrer/)
|
t-measure-probability |
149/7 |
Mathlib.lean,Mathlib/Probability/Distributions/Bernoulli.lean,Mathlib/Probability/HasLaw.lean |
3 |
4 |
['DavidLedvinka', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
1-84187 1 day ago |
2-20455 2 days ago |
7-50293 7 days |
| 31880 |
gululu996-ui author:gululu996-ui |
feat(Combinatorics/SimpleGraph/Hamiltonian): Add theorem 'IsNotHamiltonian_if_IsBridge' |
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-combinatorics
awaiting-author
|
56/1 |
Mathlib/Combinatorics/SimpleGraph/Hamiltonian.lean |
1 |
14 |
['SnirBroshi', 'github-actions', 'jcommelin'] |
nobody |
1-84125 1 day ago |
8-63931 8 days ago |
5-19213 5 days |
| 31901 |
callesonne author:callesonne |
feat(Bicategory/Subbicategory): add full subbicategories using `ObjectProperty` |
Analogously to the 1-categorical setting we construct a full subbicategory from an object property.
One could also construct locally full subbicategories using a pair of an object property and a morphism property. However then there is no way to obtain the bicategory structure by specializing from the `InducedBicategory` case. It is not clear to me if we want a full subbicategory to be specialized from this other construction, or from `InducedBicategory`.
---
- [x] depends on: #30925
[](https://gitpod.io/from-referrer/)
|
t-category-theory |
135/2 |
Mathlib.lean,Mathlib/CategoryTheory/Bicategory/Basic.lean,Mathlib/CategoryTheory/Bicategory/InducedBicategory.lean,Mathlib/CategoryTheory/Bicategory/Subbicategory.lean |
4 |
n/a |
['callesonne', 'github-actions', 'leanprover-radar', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
1-83412 1 day ago |
unknown |
unknown |
| 32385 |
kebekus author:kebekus |
feat: derivatives of meromorphic functions are meromorphic |
Show that (iterated) derivatives of meromorphic functions are again meromorphic.
---
[](https://gitpod.io/from-referrer/)
|
t-analysis |
88/2 |
Mathlib/Analysis/Calculus/Deriv/Basic.lean,Mathlib/Analysis/Calculus/FDeriv/Analytic.lean,Mathlib/Analysis/Meromorphic/Basic.lean,Mathlib/Topology/Separation/Basic.lean |
4 |
1 |
['github-actions'] |
nobody |
1-82514 1 day ago |
1-82534 1 day ago |
1-85009 1 day |
| 30582 |
RemyDegenne author:RemyDegenne |
feat: extension of a function to the closure of a submodule |
- define the closure of a set in a complete space as an `AbstractCompletion`
- add instances about submodules
- add a coercion from a submodule to its topological closure
- add induction lemmas on topological closures of submodules
- define the extension of a function on a submodule to the closure of a submodule
---
[](https://gitpod.io/from-referrer/)
|
t-topology
WIP
|
138/1 |
Mathlib/Topology/Algebra/Module/Basic.lean,Mathlib/Topology/UniformSpace/AbstractCompletion.lean |
2 |
7 |
['ADedecker', 'RemyDegenne', 'github-actions', 'mathlib4-merge-conflict-bot', 'mcdoll'] |
PatrickMassot and mcdoll assignee:PatrickMassot assignee:mcdoll |
1-82052 1 day ago |
1-82053 1 day ago |
35-55566 35 days |
| 26351 |
RemyDegenne author:RemyDegenne |
feat: covering and packing numbers of sets in a metric space |
We define covering numbers of sets in a pseudo-metric space, which are minimal cardinalities of
`ε`-covers of sets. We also define the packing number, which is the maximal cardinality of
an `ε`-separated set.
From the Brownian motion project.
---
- [x] depends on: #31537
[](https://gitpod.io/from-referrer/)
|
brownian
t-topology
awaiting-author
|
212/0 |
Mathlib.lean,Mathlib/Topology/MetricSpace/CoveringNumbers.lean |
2 |
16 |
['ADedecker', 'RemyDegenne', 'YaelDillies', 'github-actions', 'j-loreaux', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
j-loreaux assignee:j-loreaux |
1-81317 1 day ago |
1-81778 1 day ago |
45-38108 45 days |
| 32367 |
BoltonBailey author:BoltonBailey |
feat(Computability): add finEncodings for List Bool and pairs of types |
This PR contains `finEncoding`s relevant to developing complexity theory in downstream libraries. It is adapted from [this](https://leanprover.zulipchat.com/#narrow/channel/116395-maths/topic/Formalise.20the.20proposition.20P.20.E2.89.A0NP/near/451765788)[#maths > Formalise the proposition P ≠NP @ 💬](https://leanprover.zulipchat.com/#narrow/channel/116395-maths/topic/Formalise.20the.20proposition.20P.20.E2.89.A0NP/near/451765788) comment.
Co-authored-by: Daniel Weber
---
[](https://gitpod.io/from-referrer/)
|
|
58/3 |
Mathlib/Computability/Encoding.lean,Mathlib/Data/List/Basic.lean,Mathlib/Data/Sum/Basic.lean |
3 |
1 |
['github-actions'] |
nobody |
1-81287 1 day ago |
2-44754 2 days ago |
2-44731 2 days |
| 31551 |
RemyDegenne author:RemyDegenne |
feat: `gaussianReal_const_sub` |
- Add lemmas stating that if `X` is a real Gaussian random variable with mean `μ` and variance `v`, then `-X`, `X - y` and `y - X` are Gaussian with variance `v` and respective means `-μ`, `μ - y` and `y - μ`.
- Generalize this section of the file from `MeasureSpace` to `MeasurableSpace`+`Measure`
---
[](https://gitpod.io/from-referrer/)
|
t-measure-probability |
31/23 |
Mathlib/Probability/Distributions/Gaussian/Real.lean |
1 |
4 |
['EtienneC30', 'github-actions'] |
EtienneC30 assignee:EtienneC30 |
1-80835 1 day ago |
1-80884 1 day ago |
2-22673 2 days |
| 32064 |
chrisflav author:chrisflav |
feat(RingTheory/Smooth): smooth algebra over Noetherian base is flat |
Co-authored by: Judith Ludwig
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory |
324/1 |
Mathlib.lean,Mathlib/RingTheory/AdicCompletion/Algebra.lean,Mathlib/RingTheory/AdicCompletion/RingHom.lean,Mathlib/RingTheory/Ideal/Quotient/Operations.lean,Mathlib/RingTheory/Smooth/AdicCompletion.lean,Mathlib/RingTheory/Smooth/Flat.lean,docs/references.bib |
7 |
16 |
['chrisflav', 'erdOne', 'github-actions'] |
nobody |
1-80513 1 day ago |
1-80581 1 day ago |
5-29592 5 days |
| 31898 |
ntapiam author:ntapiam |
feat(LinearAlgebra/TensorAlgebra): implement HopfAlgebra for TensorAlgebra |
implementation of the natural Hopf algebra structure on the TensorAlgebra |
t-ring-theory
new-contributor
awaiting-author
|
253/0 |
Mathlib.lean,Mathlib/Algebra/FreeAlgebra.lean,Mathlib/LinearAlgebra/TensorAlgebra/Basic.lean,Mathlib/RingTheory/Bialgebra/FreeAlgebra.lean,Mathlib/RingTheory/Bialgebra/TensorAlgebra.lean,Mathlib/RingTheory/HopfAlgebra/TensorAlgebra.lean |
6 |
63 |
['YaelDillies', 'github-actions', 'kckennylau', 'ntapiam'] |
nobody |
1-79107 1 day ago |
12-27378 12 days ago |
0-63895 17 hours |
| 32389 |
LLaurance author:LLaurance |
feat(Analysis): Trigonometric identities |
`sin` and `cos` of real and complex integer multiples of π/12
---
Resolves https://github.com/leanprover-community/mathlib4/pull/28630#discussion_r2307957255
[](https://gitpod.io/from-referrer/)
|
|
174/0 |
Mathlib/Analysis/SpecialFunctions/Trigonometric/Basic.lean |
1 |
1 |
['github-actions'] |
nobody |
1-78120 1 day ago |
1-78120 1 day ago |
1-79757 1 day |
| 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
- [x] depends on: #29137
- [x] depends on: #29143
[](https://gitpod.io/from-referrer/)
|
large-import
t-measure-probability
WIP
|
1713/1 |
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 |
11 |
7 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
1-69201 1 day ago |
1-69557 1 day ago |
0-1 1 second |
| 32382 |
YaelDillies author:YaelDillies |
chore(Algebra/Order/AddGroupWithTop): golf |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
107/154 |
Mathlib/Algebra/Order/AddGroupWithTop.lean,Mathlib/Algebra/Order/GroupWithZero/Canonical.lean,Mathlib/Algebra/Order/Ring/Archimedean.lean |
3 |
1 |
['github-actions'] |
nobody |
1-65845 1 day ago |
1-65845 1 day ago |
1-85516 1 day |
| 31165 |
AntoineChambert-Loir author:AntoineChambert-Loir |
feat(LinearAlgebra/Transvection): base change of transvections |
The base change of a transvection of a module.
---
- [x] depends on: #31162
- [x] depends on: #31240
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebra
delegated
label:t-algebra$ |
60/16 |
Mathlib/LinearAlgebra/Charpoly/BaseChange.lean,Mathlib/LinearAlgebra/TensorProduct/Tower.lean,Mathlib/LinearAlgebra/Transvection.lean,Mathlib/RingTheory/TensorProduct/IsBaseChangeHom.lean |
4 |
13 |
['github-actions', 'mathlib-bors', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'ocfnash'] |
ocfnash assignee:ocfnash |
1-64362 1 day ago |
1-64362 1 day ago |
1-5284 1 day |
| 32194 |
alreadydone author:alreadydone |
feat(LinearAlgebra): more on StrongRankCondition |
Strong rank condition fails for R iff there is a copy of $R^{(\mathbb{N})}$ in some $R^n$, iff some $R^n$ has infinity rank, iff some $R^{n+1}$ has zero `finrank`. As consequences, if all $R^n$ are Noetherian or Artinian, then $R$ satisfies the strong rank condition.
To prove the first equivalence, I redeveloped a version of the ["tunnels and tailings"](https://github.com/leanprover-community/mathlib3/commit/86766851#diff-7829719aad6a9e3e617da2a7cf29dba4d55516b27e18f240eca352f4983d67b7R472-R491) construction @jcommelin and @kim-em contributed to mathlib ~4 years ago and made it work for Semiring/AddCommMonoid. The original construction was deprecated in [#12076](https://github.com/leanprover-community/mathlib4/commit/5948566497f56e1432c52d65623f1bb3c3937159) by @acmepjz and later removed, though some docstrings still remain, and I think it's now time to remove it.
Also add an instance that finite semirings satisfy the Orzech property (and therefore strong rank condition and invariant basis number).
---
- [x] depends on: #32123
[](https://gitpod.io/from-referrer/)
|
t-algebra
awaiting-author
label:t-algebra$ |
201/106 |
Mathlib/Data/Finsupp/Basic.lean,Mathlib/Data/Fintype/Card.lean,Mathlib/Data/Fintype/EquivFin.lean,Mathlib/LinearAlgebra/Dimension/StrongRankCondition.lean,Mathlib/LinearAlgebra/Finsupp/Pi.lean,Mathlib/LinearAlgebra/InvariantBasisNumber.lean,Mathlib/LinearAlgebra/LinearIndependent/Lemmas.lean,Mathlib/LinearAlgebra/Prod.lean,Mathlib/RingTheory/Artinian/Instances.lean,Mathlib/RingTheory/Artinian/Module.lean,Mathlib/RingTheory/Noetherian/Basic.lean,Mathlib/RingTheory/OrzechProperty.lean |
12 |
4 |
['alreadydone', 'eric-wieser', 'github-actions', 'mathlib4-dependent-issues-bot'] |
eric-wieser assignee:eric-wieser |
1-62631 1 day ago |
3-4374 3 days ago |
3-57583 3 days |
| 32339 |
alreadydone author:alreadydone |
chore(LinearAlgebra/Dimension): generalize and golf |
LinearAlgebra/Dimension/Finite.lean: generalize Ring/AddCommGroup to Semiring/AddCommMonoid whenever possible
LinearAlgebra/Dimension/DivisionRing.lean: generalize DivisionRing to OrzechProperty
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
81/116 |
Mathlib/LinearAlgebra/Dimension/DivisionRing.lean,Mathlib/LinearAlgebra/Dimension/Finite.lean |
2 |
1 |
['github-actions'] |
nobody |
1-62370 1 day ago |
3-21568 3 days ago |
3-21546 3 days |
| 32373 |
erdOne author:erdOne |
feat(Analysis): `HasFPowerSeriesOnBall (fun x ↦ 1 / (1 - x))` and friends |
---
[](https://gitpod.io/from-referrer/)
|
t-analysis |
141/1 |
Mathlib/Analysis/Analytic/Binomial.lean,Mathlib/Analysis/Analytic/OfScalars.lean |
2 |
1 |
['github-actions'] |
nobody |
1-61500 1 day ago |
2-32609 2 days ago |
2-32648 2 days |
| 32395 |
ADedecker author:ADedecker |
feat: specialize `[pre, post]comp_uniformConvergenceCLM` to `CompactConvergenceCLM` |
---
[](https://gitpod.io/from-referrer/)
|
t-topology |
33/5 |
Mathlib/Topology/Algebra/Module/StrongTopology.lean |
1 |
1 |
['github-actions'] |
nobody |
1-61272 1 day ago |
1-73166 1 day ago |
1-73205 1 day |
| 30880 |
themathqueen author:themathqueen |
feat(Analysis/InnerProductSpace): finite-dimensional inner product space with an algebra implies a coalgebra |
A finite-dimensional inner product space with an algebra structure also has a coalgebra structure by taking adjoints of the multiplication map and algebra map. This is implemented by providing a linear isometric equivalence between the inner product space and a normed algebra.
There is also the opposite implication, i.e., a finite-dimensional inner product space with a coalgebra structure implies an algebra where `x * y = (adjoint comul) (x ⊗ₜ y)` and `algebraMap = adjoint counit`.
Motivation:
Sometimes, in a finite-dimensional C*-algebra endowed with a faithful and positive linear functional, we will want to use this adjoint coalgebra structure. This comes up a lot in non-commutative graph theory, for example.
---
[](https://gitpod.io/from-referrer/)
|
maintainer-merge
t-analysis
awaiting-author
|
182/0 |
Mathlib.lean,Mathlib/Analysis/InnerProductSpace/Adjoint.lean,Mathlib/Analysis/InnerProductSpace/Coalgebra.lean,Mathlib/Analysis/InnerProductSpace/TensorProduct.lean,Mathlib/LinearAlgebra/TensorProduct/Associator.lean |
5 |
34 |
['github-actions', 'j-loreaux', 'mathlib4-merge-conflict-bot', 'ocfnash', 'themathqueen'] |
urkud assignee:urkud |
1-55984 1 day ago |
1-55984 1 day ago |
37-50225 37 days |
| 32381 |
YaelDillies author:YaelDillies |
chore: deprecate `ENat.not_lt_zero` in favor of `not_neg` |
---
[](https://gitpod.io/from-referrer/)
|
t-data
maintainer-merge
|
2/2 |
Mathlib/Data/ENat/Basic.lean |
1 |
11 |
['Ruben-VandeVelde', 'YaelDillies', 'b-mehta', 'github-actions', 'grunweg', 'ocfnash'] |
nobody |
1-55170 1 day ago |
1-56855 1 day ago |
1-84170 1 day |
| 32131 |
Vierkantor author:Vierkantor |
feat(scripts): count the number of tactics without a docstring |
We want to make sure every tactic is well documented. Right now, I count 33 tactics in Mathlib without any docstring at all. Add this number to the weekly technical debt metrics bot so we can track it and fix any regressions.
---
[](https://gitpod.io/from-referrer/)
|
large-import
CI
t-meta
|
68/1 |
Mathlib.lean,Mathlib/Init.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter/TacticDocumentation.lean,scripts/nolints.json,scripts/technical-debt-metrics.sh |
6 |
18 |
['Vierkantor', 'adomani', 'bryangingechen', 'github-actions'] |
joneugster assignee:joneugster |
1-55059 1 day ago |
1-55191 1 day ago |
6-72888 6 days |
| 30570 |
SnirBroshi author:SnirBroshi |
feat(Combinatorics/SimpleGraph/Connectivity/Connected): `reachabilitySet` |
Define `reachabilitySet` as the set of all pairs that have a walk between them.
`reachabilitySet` is to `Reachable` what `edgeSet` is to `Adj` (both related by `Sym2.fromRel`).
---
The main motivation is making it easier to work with the bridge definition (see `isBridge_iff_mem_edgeSet_and_notMem_reachabilitySet_deleteEdges` and `mem_edgeSet_and_mem_reachabilitySet_deleteEdges_iff_exists_isCycle_and_mem_edges` at the bottom), although I think this set is worth defining regardless.
- [x] depends on: #30542
[](https://gitpod.io/from-referrer/)
|
t-combinatorics |
61/0 |
Mathlib/Combinatorics/SimpleGraph/Connectivity/Connected.lean |
1 |
7 |
['SnirBroshi', 'b-mehta', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
kex-y assignee:kex-y |
1-53045 1 day ago |
14-1128 14 days ago |
27-54529 27 days |
| 32383 |
joelriou author:joelriou |
feat(Algebra/Homology): extensions of bifunctors to complexes preserve homotopies |
Given a `TotalComplexShape c₁ c₂ c`, a functor `F : C₁ ⥤ C₂ ⥤ D`, we show in this PR that up to homotopy the morphism `mapBifunctorMap f₁ f₂ F c` only depends on the homotopy classes of the morphism `f₁` in `HomologicalComplex C c₁` and of the morphism `f₂` in `HomologicalComplex C c₂`.
(The case of `f₁` was already done, the case of `f₂` is obtained in this PR by symmetry.)
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-category-theory
label:t-algebra$ |
118/8 |
Mathlib/Algebra/Homology/BifunctorFlip.lean,Mathlib/Algebra/Homology/BifunctorHomotopy.lean,Mathlib/Algebra/Homology/ComplexShapeSigns.lean |
3 |
1 |
['github-actions'] |
nobody |
1-52675 1 day ago |
1-85258 1 day ago |
1-85294 1 day |
| 30605 |
joelriou author:joelriou |
feat(CategoryTheory): for any filtered category, there exists a final functor from a directed poset |
In this PR, we formalize the proof by Deligne (SGA 4 I 8.1.6) that for any (small) filtered category `J`, there exists a final functor `F : α ⥤ J` where `α` is a directed partially ordered set (`IsFiltered.exists_directed`). The construction applies more generally to `κ`-filtered categories and `κ`-directed posets (`IsCardinalFiltered.exists_cardinal_directed`).
---
- [x] depends on: #31426
- [x] depends on: #31421
- [x] depends on: #31424
- [x] depends on: #30633
- [x] depends on: #30781
- [x] depends on: #30634
[](https://gitpod.io/from-referrer/)
|
t-category-theory
awaiting-author
|
304/3 |
Mathlib/CategoryTheory/Comma/Arrow.lean,Mathlib/CategoryTheory/Filtered/Basic.lean,Mathlib/CategoryTheory/Limits/Preserves/Filtered.lean,Mathlib/CategoryTheory/Presentable/Directed.lean,docs/references.bib |
5 |
10 |
['alreadydone', 'dagurtomas', 'github-actions', 'joelriou', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
dagurtomas and robin-carlier assignee:dagurtomas assignee:robin-carlier |
1-51272 1 day ago |
1-51272 1 day ago |
6-23846 6 days |
| 32406 |
JovanGerb author:JovanGerb |
feat(tauto): better error message on failure |
This PR improves the `tauto` error message. Previously, it said "tauto failed to solve some goals.", and then a separate message reported on the unsolved goals. But I think these unsolved goals are implementation details of `tauto`. So instead, the error message now says "Tactic `tauto` failed", followed by the goal on which `tauto` was run.
This change is so that `tauto` can be used as part of the `by_contra!` tactic.
---
[](https://gitpod.io/from-referrer/)
|
t-meta |
4/24 |
Mathlib/Lean/Elab/Tactic/Basic.lean,Mathlib/Tactic/Tauto.lean |
2 |
1 |
['github-actions'] |
nobody |
1-50647 1 day ago |
1-52188 1 day ago |
1-52228 1 day |
| 31711 |
joelriou author:joelriou |
feat(CategoryTheory/Sites): the category structure on the points of a site |
---
- [x] depends on: #31708
- [x] depends on: #31710
- [x] depends on: #31859
[](https://gitpod.io/from-referrer/)
|
t-category-theory |
128/3 |
Mathlib.lean,Mathlib/CategoryTheory/Sites/Point/Basic.lean,Mathlib/CategoryTheory/Sites/Point/Category.lean |
3 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
1-48726 1 day ago |
1-48778 1 day ago |
1-48756 1 day |
| 31998 |
Thmoas-Guan author:Thmoas-Guan |
feat(Algebra): localized module in `ModuleCat` |
For `ModuleCat.{v} R` and `R` being `Small.{v} R`, localized module can be canonically constructed
within `ModuleCat.{v} (Localization S)`.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
awaiting-author
label:t-algebra$ |
100/0 |
Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Localization.lean |
2 |
22 |
['Thmoas-Guan', 'dagurtomas', 'github-actions'] |
dagurtomas and kim-em assignee:kim-em assignee:dagurtomas |
1-47913 1 day ago |
1-47913 1 day ago |
9-49169 9 days |
| 32386 |
riccardobrasca author:riccardobrasca |
feat: add classical version of Hilbert 90 |
We add the classical formulation of Hilbert's theorem 90: let `L/K` be a finite Galois extension of fields such that the Galois group is cyclic generated by `σ`. Let `η` be an element of `L` of norm `1`. Then there exists `ε` such that `η = ε / σ ε`.
We also add an integral version.
Co-authored by: Andrew Yang [the.erd.one@gmail.com](mailto:the.erd.one@gmail.com)
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-number-theory
WIP
|
160/7 |
Mathlib/Algebra/BigOperators/Group/Finset/Basic.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/Hilbert90.lean |
2 |
10 |
['copilot-pull-request-reviewer', 'erdOne', 'github-actions', 'plp127', 'riccardobrasca'] |
nobody |
1-46792 1 day ago |
1-67350 1 day ago |
0-12668 3 hours |
| 31528 |
bwangpj author:bwangpj |
feat: MulAction.fixedPoints and MulAction.fixedBy under MulActionHom |
MulActionHom maps fixedPoints to fixedPoints and fixedBy to fixedBy.
---
[](https://gitpod.io/from-referrer/)
|
t-group-theory
large-import
|
22/1 |
Mathlib/GroupTheory/GroupAction/FixedPoints.lean |
1 |
9 |
['adomani', 'bwangpj', 'dagurtomas', 'github-actions', 'mathlib4-merge-conflict-bot'] |
dagurtomas assignee:dagurtomas |
1-45788 1 day ago |
1-53186 1 day ago |
20-13023 20 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 |
85/0 |
Mathlib/Algebra/BigOperators/Fin.lean,Mathlib/Algebra/BigOperators/Group/List/Basic.lean,Mathlib/Algebra/BigOperators/Group/List/Defs.lean,Mathlib/Data/Fin/Tuple/Basic.lean,Mathlib/Data/List/InsertIdx.lean |
5 |
15 |
['ShreckYe', 'bryangingechen', 'eric-wieser', 'github-actions', 'mathlib4-merge-conflict-bot'] |
bryangingechen assignee:bryangingechen |
1-43898 1 day ago |
1-43898 1 day ago |
81-32798 81 days |
| 31794 |
thorimur author:thorimur |
feat: `unusedFintypeInType` linter |
Adds an `UnusedInstancesInType` linter which suggests replacing `Fintype` instances with `Finite` or removing them.
This linter is off by default: it is turned on in #31795.
---
- [x] depends on: #31142
[](https://gitpod.io/from-referrer/)
|
|
164/5 |
Mathlib/Tactic/Linter/UnusedInstancesInType.lean,MathlibTest/UnusedInstancesInType.lean |
2 |
4 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
1-43457 1 day ago |
1-48677 1 day ago |
0-0 0 seconds |
| 31653 |
ster99 author:ster99 |
feat(MeasureTheory): Foelner filters |
Define a predicate for a filter to be Foelner. Prove that if a measure space with a G-action has a Foelner filter then there is a left-invariant finitely additive probability measure on it (amenability).
Define the maximal Foelner filter and prove that if the maximal Foelner filter is nontrivial, then the amenability condition above holds.
Closes #29213.
---
depends on : #32117.
[](https://gitpod.io/from-referrer/)
|
new-contributor
awaiting-author
|
205/0 |
Mathlib.lean,Mathlib/MeasureTheory/FoelnerFilter.lean |
2 |
39 |
['ADedecker', 'YaelDillies', 'github-actions', 'mathlib4-merge-conflict-bot', 'ster99'] |
nobody |
1-42308 1 day ago |
7-42990 7 days ago |
0-68014 18 hours |
| 32250 |
ADedecker author:ADedecker |
feat: integration against a locally integrable function as a CLM on test functions |
Aka viewing a locally integrable function as a distribution
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-analysis
|
189/0 |
Mathlib/Analysis/Distribution/ContDiffMapSupportedIn.lean,Mathlib/Analysis/Distribution/TestFunction.lean |
2 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
1-41338 1 day ago |
3-75552 3 days ago |
0-0 0 seconds |
| 30116 |
FormulaRabbit81 author:FormulaRabbit81 |
feat(Measure): proof that a relatively compact set of measures is tight |
---
[](https://gitpod.io/from-referrer/)
|
t-measure-probability
awaiting-author
|
197/2 |
Mathlib/MeasureTheory/Measure/Tight.lean |
1 |
14 |
['EtienneC30', 'github-actions', 'mathlib4-merge-conflict-bot'] |
RemyDegenne assignee:RemyDegenne |
1-40813 1 day ago |
1-40813 1 day ago |
59-65157 59 days |
| 32128 |
grunweg author:grunweg |
dev: investigate the private module linter not firing |
Only for debugging.
(1) wait for CI to rebuild everything until separablyGenerated
(2) make any modifications to the linter to dump debugging state
(3) try to find the bug with it
---
[](https://gitpod.io/from-referrer/)
|
|
406/5 |
Mathlib.lean,Mathlib/FieldTheory/Perfect.lean,Mathlib/FieldTheory/SeparablyGenerated.lean,Mathlib/Init.lean,Mathlib/RingTheory/AlgebraicIndependent/Defs.lean,Mathlib/Tactic/Linter.lean,Mathlib/Tactic/Linter/PrivateModule.lean |
7 |
3 |
['github-actions', 'grunweg'] |
nobody |
1-39184 1 day ago |
1-39205 1 day ago |
1-44953 1 day |
| 31807 |
edegeltje author:edegeltje |
feat(CategoryTheory/Cat/Basic): Turning 1- and 2-morphisms in Cat into a 1-field structure |
This PR defines `Cat.Hom` and `Cat.Hom₂`, which are 1-field structures wrapping `Functor` and `NatTrans` respectively.
In addition, it changes the `Bicategory` instance for `Cat` to use these wrappers instead.
This PR adds such definitions as `NatTrans.toCatHom2`, `Cat.Hom.toFunctor`, `Cat.Hom₂.toNatTrans`, `Cat.Hom.isoMk` as well as simp lemmas for normalizing these to operations.
---
[](https://gitpod.io/from-referrer/)
|
t-category-theory
awaiting-author
|
835/617 |
Mathlib/Algebra/Category/ModuleCat/Pseudofunctor.lean,Mathlib/AlgebraicTopology/Quasicategory/StrictBicategory.lean,Mathlib/AlgebraicTopology/SimplicialSet/HomotopyCat.lean,Mathlib/AlgebraicTopology/SimplicialSet/Nerve.lean,Mathlib/AlgebraicTopology/SimplicialSet/NerveAdjunction.lean,Mathlib/CategoryTheory/Bicategory/CatEnriched.lean,Mathlib/CategoryTheory/Bicategory/Functor/Cat.lean,Mathlib/CategoryTheory/Bicategory/Grothendieck.lean,Mathlib/CategoryTheory/Category/Cat.lean,Mathlib/CategoryTheory/Category/Cat/Adjunction.lean,Mathlib/CategoryTheory/Category/Cat/AsSmall.lean,Mathlib/CategoryTheory/Category/Cat/CartesianClosed.lean,Mathlib/CategoryTheory/Category/Cat/Limit.lean,Mathlib/CategoryTheory/Category/Cat/Op.lean,Mathlib/CategoryTheory/Category/Cat/Terminal.lean,Mathlib/CategoryTheory/Category/Grpd.lean,Mathlib/CategoryTheory/Category/Quiv.lean,Mathlib/CategoryTheory/Category/ReflQuiv.lean,Mathlib/CategoryTheory/CodiscreteCategory.lean,Mathlib/CategoryTheory/Comma/Over/Basic.lean,Mathlib/CategoryTheory/Comma/StructuredArrow/Final.lean,Mathlib/CategoryTheory/Comma/StructuredArrow/Functor.lean,Mathlib/CategoryTheory/Elements.lean,Mathlib/CategoryTheory/FiberedCategory/Grothendieck.lean,Mathlib/CategoryTheory/Filtered/Grothendieck.lean,Mathlib/CategoryTheory/Functor/KanExtension/Adjunction.lean,Mathlib/CategoryTheory/Grothendieck.lean,Mathlib/CategoryTheory/Groupoid/FreeGroupoidOfCategory.lean,Mathlib/CategoryTheory/IsomorphismClasses.lean,Mathlib/CategoryTheory/Join/Pseudofunctor.lean,Mathlib/CategoryTheory/Limits/Final.lean,Mathlib/CategoryTheory/Limits/Shapes/Grothendieck.lean,Mathlib/CategoryTheory/Monoidal/Cartesian/Cat.lean,Mathlib/CategoryTheory/SingleObj.lean,Mathlib/CategoryTheory/Sites/Descent/DescentData.lean,Mathlib/CategoryTheory/Sites/Descent/IsPrestack.lean,Mathlib/CategoryTheory/Sites/PseudofunctorSheafOver.lean,Mathlib/CategoryTheory/WithTerminal/Basic.lean,Mathlib/Order/Category/Preord.lean,Mathlib/Tactic/CategoryTheory/ToApp.lean,MathlibTest/CategoryTheory/ToApp.lean |
41 |
24 |
['callesonne', 'edegeltje', 'github-actions', 'joelriou', 'mathlib4-merge-conflict-bot'] |
nobody |
1-39159 1 day ago |
1-58046 1 day ago |
9-77991 9 days |
| 32264 |
jjtowery author:jjtowery |
feat(Bicategory): add lax slice bicategory |
---
In this PR, I define the lax slice bicategory for a lax functor over an object. I also give the change of slice strict pseudofunctor. These are from Section 7.1 of Johnson & Yau and are essential for their Whitehead theorem for bicategories (lax functor biequivalence iff essentially surjective, essentially full, and fully faithful), which I'd like to prove at some point.
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-category-theory
awaiting-author
|
527/0 |
Mathlib.lean,Mathlib/CategoryTheory/Bicategory/LaxSlice.lean |
2 |
6 |
['dagurtomas', 'github-actions', 'jjtowery'] |
dagurtomas assignee:dagurtomas |
1-37390 1 day ago |
1-39791 1 day ago |
3-50916 3 days |
| 32370 |
apnelson1 author:apnelson1 |
feat(Combinatorics/Matroid): refactor matroid supportedness tactic |
WIP refactor of the `aesop_mat` tactic that automatically proves something is a subset/member of the ground set to use `grind` rather than `aesop`.
Tactic is renamed `ground`.
---
[](https://gitpod.io/from-referrer/)
|
WIP |
173/186 |
Mathlib/Combinatorics/Matroid/Basic.lean,Mathlib/Combinatorics/Matroid/Circuit.lean,Mathlib/Combinatorics/Matroid/Closure.lean,Mathlib/Combinatorics/Matroid/Dual.lean,Mathlib/Combinatorics/Matroid/IndepAxioms.lean,Mathlib/Combinatorics/Matroid/Init.lean,Mathlib/Combinatorics/Matroid/Loop.lean,Mathlib/Combinatorics/Matroid/Minor/Contract.lean,Mathlib/Combinatorics/Matroid/Minor/Delete.lean,Mathlib/Combinatorics/Matroid/Minor/Order.lean,Mathlib/Combinatorics/Matroid/Minor/Restrict.lean,Mathlib/Combinatorics/Matroid/Rank/Cardinal.lean,Mathlib/Combinatorics/Matroid/Rank/ENat.lean,Mathlib/Combinatorics/Matroid/Rank/Finite.lean,Mathlib/RingTheory/AlgebraicIndependent/TranscendenceBasis.lean,Mathlib/Tactic/Attr/Register.lean |
16 |
7 |
['apnelson1', 'github-actions', 'leanprover-radar'] |
nobody |
1-36982 1 day ago |
2-40696 2 days ago |
0-10 10 seconds |
| 29948 |
mcdoll author:mcdoll |
feat(Analysis/Fourier): the Fourier transform on L^2 |
---
- [x] depends on: #29888
- [x] depends on: #29860
- [x] depends on: #31074
- [x] depends on: #31076
- [x] depends on: #31079
[](https://gitpod.io/from-referrer/)
|
large-import
t-analysis
|
116/5 |
Mathlib.lean,Mathlib/Analysis/Distribution/FourierSchwartz.lean,Mathlib/Analysis/Distribution/SchwartzSpace.lean,Mathlib/Analysis/Fourier/L2Space.lean,Mathlib/Analysis/Normed/Lp/SmoothApprox.lean,docs/undergrad.yaml |
6 |
4 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
1-36305 1 day ago |
2-27809 2 days ago |
2-31993 2 days |
| 32405 |
Shaddaaa author:Shaddaaa |
feat(CategoryTheory/Sites): (Co)continuity of `Over.iteratedSliceEquiv` |
Show that the `Over.iteratedSliceEquiv` functor is continuous and cocontinuous.
This contribution was created as part of the Heidelberg Lean workshop "Formalising algebraic geometry" in November 2025.
Co-authored-by: Ben Eltschig @peabrainiac
Co-authored-by: Andrew Yang @erdOne
---
[](https://gitpod.io/from-referrer/)
|
large-import
new-contributor
t-category-theory
awaiting-author
|
76/3 |
Mathlib/CategoryTheory/Sites/Equivalence.lean,Mathlib/CategoryTheory/Sites/Over.lean |
2 |
10 |
['Shaddaaa', 'dagurtomas', 'erdOne', 'github-actions'] |
nobody |
1-34006 1 day ago |
1-35333 1 day ago |
0-19390 5 hours |
| 31433 |
sinhp author:sinhp |
feat(CategoryTheory): Computable cartesian monoidal structure on slices induced by chosen pullbacks |
We provide for a category `C` with chosen pullbacks, a cartesian monoidal structure on the slice categories `Over X` for all objects `X : C`.
We also show that the functor `pullback f : Over X ⥤ Over Y` is naturally isomorphic to `toOver (Over.mk f): Over X ⥤ Over (Over.mk f)` post-composed with the iterated slice equivalence `Over (Over.mk f) ⥤ Over Y`.
This latter theorem will be crucial in relating closed objects in the slices to exponentiable morphisms in the base in `LocallyCartesianClosed.Basic.lean`
(Here `toOver` is defined to be the computable analogue of the functor `Over.star`.)
```mermaid
graph TD
A[ChosenPullbackAlong.lean] --> A'[Over.lean]
A' --> B[Sections.lean]
A --> C[ExponentiableMorphism.lean]
B --> D[Basic.lean]
C --> D
D --> E[Types.lean]
E --> F[Presheaves.lean]
D --> G[Beck-Chevalley.lean]
%% Define highlight style
classDef highlight fill:#ffe599,stroke:#d4a017,stroke-width:2px;
%% Apply to one node
class A' highlight;
```
---
- [x] depends on: #31033
[](https://gitpod.io/from-referrer/)
|
t-category-theory
awaiting-author
|
344/3 |
Mathlib.lean,Mathlib/CategoryTheory/Comma/Over/Basic.lean,Mathlib/CategoryTheory/LocallyCartesianClosed/ChosenPullbacksAlong.lean,Mathlib/CategoryTheory/LocallyCartesianClosed/Over.lean |
4 |
37 |
['dagurtomas', 'github-actions', 'joelriou', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'robin-carlier', 'sinhp'] |
robin-carlier assignee:robin-carlier |
1-31621 1 day ago |
1-32834 1 day ago |
10-69481 10 days |
| 31505 |
dsfxcimk author:dsfxcimk |
feat: Add some oangle theorems |
Add several theorems relating oriented angles and affine independence / collinearity, together with auxiliary lemmas about the equality and sign of oriented angles.
Main additions
`oangle_ne_zero_and_ne_pi_iff_not_collinear`
– An oriented angle is neither `0` nor `π` if and only if the three points are not collinear.
`affineIndependent_iff_of_oangle_eq`
– If two oriented angles are equal, then the corresponding triples of points are affinely independent simultaneously.
`not_collinear_iff_of_angle_eq`
– If two oriented angles are equal, one triple is collinear if and only if the other is.
`oangle_eq_or_eq_neg_of_angle_eq`
– The oriented angles are equal or opposite if the unoriented angles are equal.
`angle_eq_neg_of_two_zsmul_angle_eq`
– If `2 • a = 2 • b` and the signs are opposite, then `a = b + π.`
`two_zsmul_eq_iff_eq`
– Characterizes equality of doubled angles when signs are equal.
`oangle_sub_oangle_ne_pi_of_not_collinear`
– If the signs of two oriented angles are equal and the points are not collinear, their difference is not `π`. |
new-contributor
t-euclidean-geometry
awaiting-author
|
72/0 |
Mathlib/Analysis/SpecialFunctions/Trigonometric/Angle.lean,Mathlib/Geometry/Euclidean/Angle/Oriented/Affine.lean |
2 |
21 |
['dsfxcimk', 'github-actions', 'jsm28'] |
nobody |
1-29856 1 day ago |
9-58185 9 days ago |
0-50 50 seconds |
| 32411 |
mcdoll author:mcdoll |
feat(Analysis/Distribution): the bilinear pairing of Schwartz functions |
We define the bilinear pairing of Schwartz functions. Since everything is in curried form, and curried continuity and uncurried continuity are different for general TVS, we record the continuity in the left argument separately.
---
[](https://gitpod.io/from-referrer/)
|
t-analysis |
18/0 |
Mathlib/Analysis/Distribution/SchwartzSpace.lean |
1 |
n/a |
['github-actions'] |
nobody |
1-27709 1 day ago |
unknown |
unknown |
| 31395 |
peakpoint author:peakpoint |
feat(Analysis/Normed/Affine/Isometry): interpret `AffineIsometry{Map,Equiv}` as `ContinuousAffine{Map,Equiv}` |
Extracted from #27378
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-analysis
|
66/3 |
Mathlib/Analysis/Normed/Affine/Isometry.lean,Mathlib/Topology/Algebra/ContinuousAffineEquiv.lean |
2 |
14 |
['github-actions', 'j-loreaux', 'jsm28', 'mathlib4-merge-conflict-bot', 'ocfnash', 'peakpoint'] |
urkud assignee:urkud |
1-26023 1 day ago |
5-12481 5 days ago |
11-35618 11 days |
| 31425 |
robertmaxton42 author:robertmaxton42 |
feat(Topology) : implement delaborators for non-standard topology notation |
Add delaborators for unary and binary notation related to non-standard topologies in the TopologicalSpace namespace.
---
[](https://gitpod.io/from-referrer/)
|
t-topology |
104/0 |
Mathlib.lean,Mathlib/Topology/Defs/Basic.lean,Mathlib/Util/DelabNonCanonical.lean,MathlibTest/Delab/TopologicalSpace.lean |
4 |
30 |
['eric-wieser', 'github-actions', 'kckennylau', 'robertmaxton42'] |
PatrickMassot assignee:PatrickMassot |
1-26022 1 day ago |
11-4564 11 days ago |
11-35457 11 days |
| 32163 |
zhuyizheng author:zhuyizheng |
feat(MeasureTheory): interval integral is absolutely continuous |
The interval integral c..x is absolutely continuous wrt x.
Part of originally planned #29508
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-measure-probability
|
98/3 |
Mathlib/MeasureTheory/Function/AbsolutelyContinuous.lean,Mathlib/MeasureTheory/Integral/IntervalIntegral/Basic.lean |
2 |
1 |
['github-actions'] |
urkud assignee:urkud |
1-26021 1 day ago |
8-22654 8 days ago |
8-22691 8 days |
| 32190 |
vihdzp author:vihdzp |
chore(Algebra/Order/Ring/Archimedean): generalize theorems to `OrderHomClass` + `RingHomClass` |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
16/12 |
Mathlib/Algebra/Order/Hom/Ring.lean,Mathlib/Algebra/Order/Ring/Archimedean.lean |
2 |
1 |
['github-actions'] |
alreadydone assignee:alreadydone |
1-26020 1 day ago |
7-39941 7 days ago |
7-39976 7 days |
| 31732 |
fbarroero author:fbarroero |
feat(NumberTheory/MahlerMeasure.lean): Northcott's Theorem |
In this file we prove Northcott's Theorem
```
theorem card_mahlerMeasure_le_prod (n : ℕ) (B : ℝ≥0) :
Nat.card {p : ℤ[X] | p.natDegree ≤ n ∧ (p.map (Int.castRingHom ℂ)).mahlerMeasure ≤ B} ≤
∏ i : Fin (n + 1), (2 * ⌊n.choose i * B⌋₊ + 1)
```
---
- [x] depends on: #31617
[](https://gitpod.io/from-referrer/)
|
t-number-theory |
103/0 |
Mathlib.lean,Mathlib/Data/Set/Card.lean,Mathlib/NumberTheory/MahlerMeasure.lean |
3 |
13 |
['MichaelStollBayreuth', 'copilot-pull-request-reviewer', 'fbarroero', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
MichaelStollBayreuth assignee:MichaelStollBayreuth |
1-5234 1 day ago |
1-5234 1 day ago |
7-8796 7 days |
| 31247 |
rudynicolop author:rudynicolop |
feat(Computability/DFA): add DFA complement, union, and intersection |
Add theorems for DFA complement, union, and intersection closure, and prove that regular languages are closed under complement, union, and intersection.
---
Note there's a [zulip discussion](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Regular.20languages.3A.20the.20review.20queue/with/553522644) regarding PRs for regular languages (also tracked in #24205). Admittedly, this is yet another PR, and this may prove obsolete if other PRs are merged first. In particular, this PR competes with #20238 and #15651.
[](https://gitpod.io/from-referrer/)
|
t-computability
new-contributor
awaiting-author
|
135/5 |
Mathlib/Computability/DFA.lean,Mathlib/Computability/Language.lean |
2 |
52 |
['YaelDillies', 'ctchou', 'github-actions', 'mathlib4-merge-conflict-bot', 'rudynicolop', 'staroperator'] |
nobody |
1-2868 1 day ago |
3-5890 3 days ago |
26-16276 26 days |
| 32254 |
YaelDillies author:YaelDillies |
feat(Algebra/MonoidAlgebra): congruence isomorphisms |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
118/12 |
Mathlib/Algebra/MonoidAlgebra/Lift.lean,Mathlib/Algebra/MonoidAlgebra/MapDomain.lean |
2 |
16 |
['YaelDillies', 'eric-wieser', 'github-actions'] |
nobody |
1-992 1 day ago |
3-2637 3 days ago |
5-35859 5 days |
| 32398 |
YaelDillies author:YaelDillies |
chore(Algebra/MonoidAlgebra): use `to_additive` more |
Using Jovan's new `dont_translate` syntax, we can tag much more of the `MonoidAlgebra` API with `to_additive`.
A few points:
1. `to_additive` currently doesn't support the destructing `have` syntax, because it generates an auxiliary `match` statement. The corresponding `obtain` syntax is fine though.
2. `AddMonoidAlgebra.opRingEquiv` and `MonoidAlgebra.opRingEquiv` were not the same statement (up to additivisation): The first assumed commutativity of the base monoid to get rid of an `AddOpposite` in the RHS. Using `to_additive` makes the type signatures align, at the cost of some shuffling around in later files. This shuffling around will become trivial after #32254.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
107/233 |
Mathlib/Algebra/MonoidAlgebra/Module.lean,Mathlib/Algebra/MonoidAlgebra/NoZeroDivisors.lean,Mathlib/Algebra/MonoidAlgebra/Opposite.lean,Mathlib/Algebra/MonoidAlgebra/Support.lean,Mathlib/RingTheory/Polynomial/Opposites.lean |
5 |
6 |
['JovanGerb', 'YaelDillies', 'github-actions'] |
nobody |
0-83425 23 hours ago |
0-83425 23 hours ago |
0-86225 23 hours |
| 32423 |
joelriou author:joelriou |
feat(CategoryTheory): more preservation properties of functors |
We consider the preservation of a limit or a colimit as an `ObjectProperty` in the category of functors.
---
[](https://gitpod.io/from-referrer/)
|
t-category-theory |
66/1 |
Mathlib/CategoryTheory/ObjectProperty/FunctorCategory/PreservesLimits.lean |
1 |
1 |
['github-actions'] |
nobody |
0-81328 22 hours ago |
0-81399 22 hours ago |
0-81376 22 hours |
| 32356 |
YuvalFilmus author:YuvalFilmus |
feat(Arsinh): add arcosh |
Defined arcosh and showed that it is inverse to cosh over the appropriate domains.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-analysis
awaiting-author
|
259/1 |
Mathlib.lean,Mathlib/Analysis/SpecialFunctions/Arcosh.lean,Mathlib/Analysis/SpecialFunctions/Arsinh.lean |
3 |
14 |
['LLaurance', 'YuvalFilmus', 'b-mehta', 'github-actions', 'j-loreaux'] |
j-loreaux assignee:j-loreaux |
0-80540 22 hours ago |
2-49930 2 days ago |
0-9694 2 hours |
| 31503 |
Scarlett-le author:Scarlett-le |
feat(Geometry/Euclidean/PerpBisector): add distance inequalities for Sbtw with perpendicularity |
This PR adds two theorems about distance relationships when points satisfy strict betweenness (`Sbtw`) and perpendicularity conditions:
### New theorems
- `dist_lt_of_sbtw_of_inner_eq_zero`: If `b` is strictly between `a` and `c`, and `p - a` is perpendicular to `b - a`, then `dist p b < dist p c`.
- `dist_lt_of_sbtw_of_mem_perpBisector`: If `p` lies on the perpendicular bisector of `ab` and `b` is strictly between `a` and `c`, then `dist p b < dist p c`. |
new-contributor
t-euclidean-geometry
awaiting-author
|
80/0 |
Mathlib/Geometry/Euclidean/PerpBisector.lean |
1 |
7 |
['Scarlett-le', 'github-actions', 'jsm28', 'mathlib4-merge-conflict-bot'] |
jsm28 assignee:jsm28 |
0-80096 22 hours ago |
9-41328 9 days ago |
8-50449 8 days |
| 32218 |
mkaratarakis author:mkaratarakis |
feat: lemmas about the `House` of an algebraic number |
Lemmas missing for the formalisation of the proof of the Gelfond–Schneider theorem
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-number-theory
awaiting-author
|
189/38 |
Mathlib/NumberTheory/NumberField/House.lean |
1 |
17 |
['github-actions', 'jcommelin', 'mkaratarakis'] |
jcommelin assignee:jcommelin |
0-78128 21 hours ago |
2-81305 2 days ago |
3-60402 3 days |
| 32426 |
kebekus author:kebekus |
doc: uniformize language |
Uniformize the language in docstrings referring to the three main functions of value distribution theory.
---
This PR is based on a suggestion of @j-loreaux during the review of a previous PR.
[](https://gitpod.io/from-referrer/)
|
t-analysis |
64/64 |
Mathlib/Analysis/Complex/ValueDistribution/CharacteristicFunction.lean,Mathlib/Analysis/Complex/ValueDistribution/CountingFunction.lean |
2 |
1 |
['github-actions'] |
nobody |
0-73617 20 hours ago |
0-74189 20 hours ago |
0-0 0 seconds |
| 32215 |
jonasvanderschaaf author:jonasvanderschaaf |
feat(ModelTheory/Types): Construct a topology on CompleteType and prove the space is compact |
---
- [x] depends on: #32213
[](https://gitpod.io/from-referrer/)
|
new-contributor |
150/0 |
Mathlib.lean,Mathlib/ModelTheory/Topology/Types.lean,Mathlib/ModelTheory/Types.lean,Mathlib/Tactic/Linter/DirectoryDependency.lean,Mathlib/Topology/Compactness/Compact.lean |
5 |
7 |
['Vierkantor', 'github-actions', 'jonasvanderschaaf', 'mathlib4-dependent-issues-bot', 'plp127'] |
nobody |
0-72692 20 hours ago |
2-67277 2 days ago |
3-48156 3 days |
| 32422 |
kim-em author:kim-em |
fix(Linter): deprecated module linter now fires for public/meta imports |
## Summary
- Fixed `getImportIds` in `Header.lean` to recognize all import variants from the new module system
- The pattern now matches `public import`, `meta import`, `public meta import`, and `import all` in addition to plain `import`
- Added test files to verify the linter fires correctly for all import variants
## Background
The deprecated module linter was not warning when using `public import` for a deprecated module. This was because `getImportIds` used a syntax pattern that only matched plain `import $n`, missing the optional `public`, `meta`, and `all` modifiers introduced in the new module system.
Reported on Zulip: https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Mathlib.20has.20moved.20to.20the.20new.20module.20system/near/561825752
## Test plan
- [x] `lake build MathlibTest.DeprecatedModuleTest` (original test still passes)
- [x] `lake build MathlibTest.DeprecatedModulePublicTest` (new test for `public import`)
- [x] `lake build MathlibTest.DeprecatedModuleMetaTest` (new test for `meta import`)
- [x] `lake build MathlibTest.DeprecatedModulePublicMetaTest` (new test for `public meta import`)
🤖 Prepared with Claude Code |
t-linter
awaiting-author
|
62/1 |
Mathlib/Tactic/Linter/Header.lean,MathlibTest/DeprecatedModuleMetaTest.lean,MathlibTest/DeprecatedModuleNew.lean,MathlibTest/DeprecatedModulePublicMetaTest.lean,MathlibTest/DeprecatedModulePublicTest.lean |
5 |
3 |
['Vierkantor', 'github-actions', 'grunweg'] |
nobody |
0-70933 19 hours ago |
0-70933 19 hours ago |
0-11260 3 hours |
| 32353 |
ADedecker author:ADedecker |
feat: define the space of distributions |
---
[](https://gitpod.io/from-referrer/)
|
maintainer-merge
t-analysis
awaiting-author
|
219/0 |
Mathlib.lean,Mathlib/Analysis/Distribution/Distribution.lean,docs/references.bib |
3 |
n/a |
['ADedecker', 'AntoineChambert-Loir', 'faenuccio', 'github-actions', 'grunweg', 'mathlib4-merge-conflict-bot', 'mcdoll'] |
nobody |
0-68860 19 hours ago |
unknown |
unknown |
| 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
awaiting-author
|
6/1 |
Mathlib/Topology/Algebra/Module/ModuleTopology.lean |
1 |
9 |
['github-actions', 'j-loreaux', 'kbuzzard', 'leanprover-bot', 'ocfnash'] |
ocfnash assignee:ocfnash |
0-66318 18 hours ago |
67-64682 2 months ago |
25-3547 25 days |
| 31478 |
BGuillemet author:BGuillemet |
feat(CategoryTheory/Sites): `uliftYoneda` for sheaves over a subcanonical topology |
Add that `GrothendieckTopology.uliftYoneda` is fully faithful.
Add the (functorial) Yoneda lemma for sheaves, for both `yoneda` and `uliftYoneda`.
---
- [x] depends on: #27821
- [x] depends on: #31538
[](https://gitpod.io/from-referrer/)
|
t-category-theory |
88/1 |
Mathlib/CategoryTheory/Sites/Canonical.lean,Mathlib/CategoryTheory/Sites/Subcanonical.lean,Mathlib/CategoryTheory/Sites/Whiskering.lean |
3 |
13 |
['BGuillemet', 'dagurtomas', 'github-actions', 'joelriou', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
0-66165 18 hours ago |
0-66165 18 hours ago |
2-2257 2 days |
| 31862 |
erdOne author:erdOne |
chore: unify `LocalizedModule` and `OreLocalization` |
We redefine `LocalizedModule` to be an abbrev of `OreLocalization S M` so that localization of a ring and localization of a module is now defeq. This is very useful to unify downstream constructions, in particular `ModuleCat.tilde` and `Spec.structureSheaf`.
Some of the declarations are switched to reducible to avoid diamonds.
This causes a significant performance regression, most notabaly in `Mathlib/AlgebraicGeometry/AffineSpace.lean`.
We shall investigate if there are ways to improve performances. For example by introducing
typeclasses to unify the two constructions on this and `LocalizedModule`, or by marking some
downstream constructions (e.g. `Spec.structureSheaf`) as irreducible.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
234/210 |
Mathlib/Algebra/Module/LocalizedModule/Basic.lean,Mathlib/AlgebraicGeometry/Modules/Tilde.lean,Mathlib/AlgebraicGeometry/Restrict.lean,Mathlib/GroupTheory/DivisibleHull.lean,Mathlib/GroupTheory/OreLocalization/Basic.lean,Mathlib/GroupTheory/OreLocalization/OreSet.lean,Mathlib/RingTheory/Localization/BaseChange.lean,Mathlib/RingTheory/OreLocalization/Ring.lean,Mathlib/RingTheory/TensorProduct/Nontrivial.lean,MathlibTest/Algebra/Module/LocalizedModule.lean |
10 |
73 |
['alreadydone', 'chrisflav', 'erdOne', 'github-actions', 'jcommelin', 'leanprover-bot', 'leanprover-radar', 'mattrobball', 'riccardobrasca', 'wwylele'] |
mariainesdff assignee:mariainesdff |
0-65323 18 hours ago |
0-65323 18 hours ago |
14-33420 14 days |
| 30089 |
loefflerd author:loefflerd |
feat(NumberTheory/ModularForms): Bounds on modular forms and q-expansion coeffs |
Show that the q-expansion coefficients of a weight k modular form grow like `n ^ k`, and like `n ^ (k / 2)` for cusp forms.
---
This is a "blockbuster" PR from which many smaller chunks will be carved off for review and submission. The first in the series are the following:
- [x] depends on: #29743
- [x] depends on: #30475
- [x] depends on: #30461
- [ ] depends on: #30471
- [ ] depends on: #30512
- [ ] depends on: #30648
[](https://gitpod.io/from-referrer/)
|
t-number-theory
WIP
|
943/94 |
Mathlib.lean,Mathlib/Analysis/Complex/CauchyIntegral.lean,Mathlib/NumberTheory/ModularForms/Basic.lean,Mathlib/NumberTheory/ModularForms/Bounds.lean,Mathlib/NumberTheory/ModularForms/Cusps.lean,Mathlib/NumberTheory/ModularForms/Identities.lean,Mathlib/NumberTheory/ModularForms/LevelOne.lean,Mathlib/NumberTheory/ModularForms/Petersson.lean,Mathlib/NumberTheory/ModularForms/QExpansion.lean,Mathlib/Topology/Algebra/Order/ArchimedeanDiscrete.lean |
10 |
n/a |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
0-64298 17 hours ago |
unknown |
unknown |
| 32077 |
artie2000 author:artie2000 |
feat(Algebra/Order/Ring/Ordering): ring ordering constructions |
* add operations on ring preorderings: intersection, bottom element, union (on directed set), map, comap
* prove how being an ordering and the support interact with each of these operations
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebra
awaiting-author
label:t-algebra$ |
347/2 |
Mathlib/Algebra/Order/Ring/Ordering/Basic.lean |
1 |
40 |
['YaelDillies', 'artie2000', 'github-actions', 'vihdzp'] |
mattrobball assignee:mattrobball |
0-64077 17 hours ago |
4-36300 4 days ago |
4-62827 4 days |
| 32424 |
joelriou author:joelriou |
feat(CategoryTheory): the Yoneda embedding for a locally small category |
Let `C` be a locally `w`-small category. We define the Yoneda embedding `shrinkYoneda : C ⥤ Cᵒᵖ ⥤ Type w`.
---
[](https://gitpod.io/from-referrer/)
|
t-category-theory |
130/0 |
Mathlib.lean,Mathlib/CategoryTheory/ShrinkYoneda.lean |
2 |
1 |
['github-actions'] |
nobody |
0-63396 17 hours ago |
0-80804 22 hours ago |
0-80782 22 hours |
| 30333 |
paulorauber author:paulorauber |
feat(Probability): definition of trajMeasure |
A definition of `trajMeasure` and some basic lemmas.
In the context of the Ionescu-Tulcea theorem, `trajMeasure μ₀ κ` corresponds to the distribution of the trajectory obtained by starting with the distribution `μ₀` and then iterating the kernels `κ`.
Lemmas `partialTraj_compProd_kernel_eq_traj_map` and `traj_map_eq_kernel` are attributable to @EtienneC30 and some definitions borrow code from @RemyDegenne , who also improved the code considerably. Please let me know if you would like to be co-authors in this pull request.
From the LeanBandits project.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-measure-probability
awaiting-author
|
81/2 |
Mathlib/Order/Interval/Finset/Basic.lean,Mathlib/Order/Interval/Finset/Nat.lean,Mathlib/Probability/Kernel/IonescuTulcea/PartialTraj.lean,Mathlib/Probability/Kernel/IonescuTulcea/Traj.lean |
4 |
25 |
['EtienneC30', 'RemyDegenne', 'github-actions', 'mathlib4-merge-conflict-bot', 'paulorauber'] |
EtienneC30 assignee:EtienneC30 |
0-63129 17 hours ago |
0-78448 21 hours ago |
7-65345 7 days |
| 30213 |
SnirBroshi author:SnirBroshi |
feat(Data/List/GetD): golf and add lemmas for `get` and `getElem?` |
---
[](https://gitpod.io/from-referrer/)
|
t-data
new-contributor
|
17/15 |
Mathlib/Data/List/GetD.lean |
1 |
23 |
['SnirBroshi', 'eric-wieser', 'github-actions', 'kim-em', 'themathqueen'] |
kim-em assignee:kim-em |
0-62757 17 hours ago |
6-24439 6 days ago |
57-29739 57 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
t-dynamics
awaiting-author
|
74/10 |
Mathlib/Dynamics/PeriodicPts/Defs.lean,Mathlib/Dynamics/PeriodicPts/Lemmas.lean,Mathlib/GroupTheory/OrderOfElement.lean |
3 |
13 |
['ShreckYe', 'dupuisf', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
dupuisf assignee:dupuisf |
0-62587 17 hours ago |
0-62587 17 hours ago |
74-34034 74 days |
| 25143 |
chrisflav author:chrisflav |
feat(RingTheory): smooth algebras have smooth Noetherian models |
Co-authored by: Judith Ludwig
---
- [x] depends on: #24794
[](https://gitpod.io/from-referrer/)
|
t-ring-theory |
270/3 |
Mathlib.lean,Mathlib/Algebra/MvPolynomial/Eval.lean,Mathlib/RingTheory/Ideal/Cotangent.lean,Mathlib/RingTheory/MvPolynomial/Homogeneous.lean,Mathlib/RingTheory/Smooth/NoetherianDescent.lean |
5 |
8 |
['chrisflav', 'erdOne', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
erdOne assignee:erdOne |
0-61439 17 hours ago |
5-61427 5 days ago |
4-34240 4 days |
| 31161 |
AntoineChambert-Loir author:AntoineChambert-Loir |
feat(RingTheory/MvPolynomial/IrrQuadratic): irreducibility of sum X_i Y_i |
For $n\geq 2$, the polynomial $$\sum_{i=1}^n X_i Y_i$$ is irreducible.
This was used in the initial proof that the transvections have determinant 1. Now,
a more general result is proved there and this PR is no more needed.
I believe that it remains of independent interest (irreducibility of quadrics in algebraic geometry) but the maintainers might want that the general one.
---
- [ ] depends on: #32226
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
awaiting-author
|
161/0 |
Mathlib.lean,Mathlib/Algebra/Polynomial/RingDivision.lean,Mathlib/RingTheory/MvPolynomial/IrrQuadratic.lean |
3 |
35 |
['AntoineChambert-Loir', 'github-actions', 'jcommelin', 'joelriou', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'ocfnash'] |
joelriou assignee:joelriou |
0-61099 16 hours ago |
0-61099 16 hours ago |
27-18525 27 days |
| 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
---
- [x] depends on: #27416
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebra
label:t-algebra$ |
247/6 |
Mathlib/RingTheory/Regular/Category.lean,Mathlib/RingTheory/Regular/Depth.lean |
2 |
n/a |
['Thmoas-Guan', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
0-60338 16 hours ago |
unknown |
unknown |
| 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
|
16/0 |
Mathlib/Data/ENat/Basic.lean |
1 |
14 |
['Ruben-VandeVelde', 'Thmoas-Guan', 'alreadydone', 'erdOne', 'github-actions', 'pechersky', 'urkud'] |
pechersky assignee:pechersky |
0-60237 16 hours ago |
7-3124 7 days ago |
37-82680 37 days |
| 32429 |
erdOne author:erdOne |
feat(RingTheory): `IsIntegrallyClosed R[X]` |
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory |
279/3 |
Mathlib.lean,Mathlib/RingTheory/IntegralClosure/IntegrallyClosed.lean,Mathlib/RingTheory/IntegralClosure/IsIntegral/AlmostIntegral.lean,Mathlib/RingTheory/Polynomial/IsIntegral.lean |
4 |
1 |
['github-actions'] |
nobody |
0-60216 16 hours ago |
0-60216 16 hours ago |
0-60374 16 hours |
| 28682 |
Thmoas-Guan author:Thmoas-Guan |
feat(RingTheory): definition of regular local ring |
In this PR, we give the definition of regular local ring.
The class `IsRegularLocalRing` is defined as `(maximalIdeal R).spanFinrank = ringKrullDim R`
We also established the lemma `IsRegularLocalRing.iff_finrank_cotangentSpace` proving this definition is equivalent to the cotangent space version.
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
awaiting-author
|
122/0 |
Mathlib.lean,Mathlib/RingTheory/RegularLocalRing/Defs.lean |
2 |
37 |
['Thmoas-Guan', 'chrisflav', 'github-actions', 'mathlib4-merge-conflict-bot', 'mbkybky'] |
chrisflav assignee:chrisflav |
0-60101 16 hours ago |
15-2215 15 days ago |
1-63449 1 day |
| 29937 |
Thmoas-Guan author:Thmoas-Guan |
feat(RingTheory): `ringKrullDim` of quotient via supportDim |
In this PR, we establish some lemma about `ringKrullDim` of quotient via lemmas of `supportDim`.
Co-authored-by: Yongle Hu @mbkybky
---
- [ ] depends on: #26219
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
awaiting-author
|
290/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/Support.lean |
8 |
4 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
0-60089 16 hours ago |
24-57975 24 days ago |
0-8336 2 hours |
| 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
awaiting-author
|
306/100 |
Mathlib.lean,Mathlib/Analysis/ODE/Basic.lean,Mathlib/Analysis/ODE/Transform.lean,Mathlib/Geometry/Manifold/IntegralCurve/Basic.lean,Mathlib/Geometry/Manifold/IntegralCurve/Transform.lean |
5 |
8 |
['github-actions', 'grunweg', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'sgouezel'] |
sgouezel assignee:sgouezel |
0-58550 16 hours ago |
0-58550 16 hours ago |
86-36467 86 days |
| 32430 |
YaelDillies author:YaelDillies |
chore: delete `Units.mulDistribMulAction'` |
This instance was intended a strengthening of `Units.mulAction'`, but in fact its conditions are so strong that it (almost) never applies! Indeed, this instance assumes both `MulDistribMulAction G M`, meaning `∀ (g : G) (m₁ m₂ : M), g • (m₁ * m₂) = g • m₁ * g • m₂`, and `SMulCommClass G M M` meaning `∀ (g : G) (m₁ m₂ : M), g • (m₁ * m₂) = m₁ * g • m₂`. In particular, if `M` is cancellative, then we obtain `∀ (g : G) (m : M), g • m = m`, i.e. the action is trivial!
The instance was added in leanprover-community/mathlib3#10480, apparently with no motivation beyond square-filling of instances.
[Zulip](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/MulDistribMulAction.20instances)
---
[](https://gitpod.io/from-referrer/)
|
bench-after-CI
t-algebra
label:t-algebra$ |
13/9 |
Mathlib/Algebra/GroupWithZero/Action/Units.lean |
1 |
1 |
['github-actions'] |
nobody |
0-57322 15 hours ago |
0-57322 15 hours ago |
0-57935 16 hours |
| 31508 |
FLDutchmann author:FLDutchmann |
feat(Tactic): `algebra` tactic. |
Implement tactic for normalizing expressions in an algebra over a ring. Handles all of the normal ring operations as well as scalar multiplication over a fixed base ring.
The core of this tactic is used by a larger suite of tactics (see #30374).
---
- [ ] depends on: #31506
For full disclosure, most of the lemma statements in `Lemmas.lean` were generated by an LLM.
[](https://gitpod.io/from-referrer/)
|
t-meta
awaiting-author
|
1565/0 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Algebra/Basic.lean,Mathlib/Tactic/Algebra/Lemmas.lean,MathlibTest/Algebra.lean,scripts/noshake.json |
6 |
12 |
['FLDutchmann', 'Vierkantor', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
Vierkantor assignee:Vierkantor |
0-57238 15 hours ago |
0-57770 16 hours ago |
9-83430 9 days |
| 30758 |
Timeroot author:Timeroot |
chore: tag abs_inv and abs_div with grind= |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
awaiting-author
label:t-algebra$ |
2/1 |
Mathlib/Algebra/Order/Field/Basic.lean |
1 |
n/a |
['github-actions'] |
nobody |
0-56269 15 hours ago |
unknown |
unknown |
| 28100 |
themathqueen author:themathqueen |
feat(LinearAlgebra/GeneralLinearGroup): algebra automorphisms in endomorphisms are inner |
Characterization of automorphisms in endomorphisms of vector spaces: for any algebra automorphism `f : End R V ≃ₐ[R] End R V`, there exists a linear isomorphism `T` such that `f a = T.conj a = T ∘ a ∘ T.symm` for all `a`. This does not suppose finite-dimensionality.
---
Technically used Aristotle for showing that `T` is injective (out of curiosity) :) (added as co-author)
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
107/12 |
Mathlib.lean,Mathlib/Algebra/Algebra/Equiv.lean,Mathlib/Algebra/Module/LinearMap/End.lean,Mathlib/FieldTheory/SplittingField/Construction.lean,Mathlib/LinearAlgebra/FreeModule/Basic.lean,Mathlib/LinearAlgebra/FreeModule/Norm.lean,Mathlib/LinearAlgebra/GeneralLinearGroup/AlgEquiv.lean,Mathlib/LinearAlgebra/Matrix/ToLin.lean,Mathlib/RingTheory/LocalRing/Module.lean |
9 |
56 |
['Whysoserioushah', 'eric-wieser', 'github-actions', 'hrmacbeth', 'kckennylau', 'mathlib4-merge-conflict-bot', 'themathqueen'] |
eric-wieser and hrmacbeth assignee:eric-wieser assignee:hrmacbeth |
0-55434 15 hours ago |
6-50992 6 days ago |
67-71355 67 days |
| 32364 |
Ruben-VandeVelde author:Ruben-VandeVelde |
feat: lemmas about bernoulli |
A step towards Euler-Maclaurin.
---
[](https://gitpod.io/from-referrer/)
|
t-analysis
t-number-theory
awaiting-author
|
227/7 |
Mathlib.lean,Mathlib/Analysis/Calculus/ContDiff/Polynomial.lean,Mathlib/NumberTheory/Bernoulli.lean,Mathlib/NumberTheory/ZetaValues.lean |
4 |
5 |
['github-actions', 'loefflerd'] |
nobody |
0-54694 15 hours ago |
0-54694 15 hours ago |
1-79608 1 day |
| 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.
- Use `TopologicalSpace.pseudoMetrizableSpaceUniformity` to endow a pseudometrizable space with a compatible uniformity,
and use `TopologicalSpace.pseudoMetrizableSpaceUniformity_countably_generated` to show that this is countably generated.
- `TopologicalSpace.pseudoMetrizableSpacePseudoMetric` and `TopologicalSpace.metrizableSpaceMetric` have been moved to `Mathlib/Topology/Metrizable/Uniformity.lean`.
See also #2032
---
[](https://gitpod.io/from-referrer/)
|
t-topology
awaiting-author
|
128/99 |
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 |
6 |
29 |
['github-actions', 'j-loreaux', 'jcommelin', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'mathlib4-merge-conflict-bot', 'plp127', 'urkud', 'vihdzp'] |
urkud assignee:urkud |
0-54262 15 hours ago |
9-8021 9 days ago |
109-56486 109 days |
| 32432 |
YaelDillies author:YaelDillies |
feat: `MulDistribMulAction M Nˣ` instance |
From ClassFieldTheory
[Zulip](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/MulDistribMulAction.20instances)
---
[](https://gitpod.io/from-referrer/)
|
CFT
t-algebra
label:t-algebra$ |
28/0 |
Mathlib/Algebra/Group/Action/Units.lean |
1 |
1 |
['github-actions'] |
nobody |
0-53961 14 hours ago |
0-53961 14 hours ago |
0-56383 15 hours |
| 32433 |
YaelDillies author:YaelDillies |
feat: an irreducible element of a submonoid isn't zero |
From ClassFieldTheory
---
[](https://gitpod.io/from-referrer/)
|
CFT
t-algebra
label:t-algebra$ |
4/0 |
Mathlib/Algebra/GroupWithZero/NonZeroDivisors.lean |
1 |
1 |
['github-actions'] |
nobody |
0-53873 14 hours ago |
0-53947 14 hours ago |
0-53926 14 hours |
| 32428 |
sven-manthe author:sven-manthe |
feat(Algebra): add Subsemigroup.op |
the file Subsemigroup.MulOpposite is analogous to Submonoid.MulOpposite. Also add trivial lemmas on relation with monoids and groups in the corresponding file
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
199/4 |
Mathlib.lean,Mathlib/Algebra/Group/Subgroup/MulOpposite.lean,Mathlib/Algebra/Group/Submonoid/MulOpposite.lean,Mathlib/Algebra/Group/Subsemigroup/MulOpposite.lean |
4 |
1 |
['github-actions'] |
nobody |
0-53344 14 hours ago |
0-65390 18 hours ago |
0-65426 18 hours |
| 32434 |
YaelDillies author:YaelDillies |
feat(Algebra/Homology): miscellaneous lemmas |
From ClassFieldTheory
---
[](https://gitpod.io/from-referrer/)
|
CFT
t-algebra
label:t-algebra$ |
21/0 |
Mathlib/Algebra/Homology/ShortComplex/Exact.lean,Mathlib/CategoryTheory/Abelian/Exact.lean |
2 |
1 |
['github-actions'] |
nobody |
0-52891 14 hours ago |
0-52961 14 hours ago |
0-52939 14 hours |
| 31717 |
thorimur author:thorimur |
chore: refactor `Type*` and `Sort*` to use `mkFreshLevelParam` |
Uses the API for creating new level parameters introduced in #30797.
---
- [ ] depends on: #30797
[](https://gitpod.io/from-referrer/)
|
large-import
t-meta
|
4/7 |
Mathlib/Tactic/TypeStar.lean |
1 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
0-52437 14 hours ago |
0-52437 14 hours ago |
3-7140 3 days |
| 29362 |
stepanholub author:stepanholub |
feat(Data/List): periods of lists; prove the Periodicity Lemma |
Add the concept of the period of a List (word, sequence) which is missing, and prove its basic nontrivial property describing under which conditions list can have two periods known as the Periodicity Lemma (aka Fine-Wilf Theorem).
---
|
t-data
new-contributor
|
240/0 |
Mathlib.lean,Mathlib/Data/List/PeriodicityLemma.lean |
2 |
139 |
['Ruben-VandeVelde', 'Timeroot', 'fpvandoorn', 'github-actions', 'jcommelin', 'madvorak', 'mathlib4-merge-conflict-bot', 'plp127', 'stepanholub', 'wwylele'] |
pechersky assignee:pechersky |
0-51633 14 hours ago |
0-53816 14 hours ago |
83-16640 83 days |
| 32435 |
YaelDillies author:YaelDillies |
chore(Algebra/Module): make select `Module` assumptions |
This solves a thorny issue that we have when working with homological algebra: an element `X : ModuleCat ℤ` by construction contain the data of two (propeq) `Module ℤ X` instances. Instead of fighting typeclasses at the point of use, it is enough to make the `Module ℤ X` assumptions that can be inferred from other arguments actually be inferred by unification, rather than filled in with typeclass search. This PR does precisely that for the handful of definitions that are particularly problematic for the purpose of CFT.
This is not unlike the status of `MeasurableSpace` in the measure theory library.
From ClassFieldTheory
---
[](https://gitpod.io/from-referrer/)
|
CFT
t-algebra
label:t-algebra$ |
22/15 |
Mathlib/Algebra/Module/Equiv/Basic.lean,Mathlib/Algebra/Module/Equiv/Defs.lean,Mathlib/Algebra/Module/LinearMap/Defs.lean |
3 |
1 |
['github-actions'] |
nobody |
0-51360 14 hours ago |
0-51438 14 hours ago |
0-51416 14 hours |
| 32427 |
YaelDillies author:YaelDillies |
refactor(Algebra/Algebra): genericise algebra instances for subsemirings |
From ClassFieldTheory
---
[](https://gitpod.io/from-referrer/)
|
CFT
t-algebra
label:t-algebra$ |
49/65 |
Mathlib/Algebra/Algebra/Basic.lean,Mathlib/Algebra/Algebra/Subalgebra/Basic.lean,Mathlib/Algebra/Algebra/Subalgebra/Tower.lean,Mathlib/Algebra/DirectSum/Internal.lean,Mathlib/Analysis/Normed/Unbundled/SpectralNorm.lean,Mathlib/NumberTheory/Cyclotomic/Basic.lean,Mathlib/NumberTheory/NumberField/CMField.lean,Mathlib/NumberTheory/Padics/PadicIntegers.lean,Mathlib/RingTheory/Algebraic/Integral.lean,Mathlib/RingTheory/Algebraic/MvPolynomial.lean,Mathlib/RingTheory/Extension/Presentation/Core.lean,Mathlib/RingTheory/IntegralClosure/IntegralRestrict.lean,Mathlib/RingTheory/LocalRing/LocalSubring.lean,Mathlib/RingTheory/Polynomial/Basic.lean,Mathlib/RingTheory/Valuation/AlgebraInstances.lean,Mathlib/RingTheory/Valuation/Integers.lean |
16 |
1 |
['github-actions'] |
nobody |
0-50725 14 hours ago |
0-71918 19 hours ago |
0-71897 19 hours |
| 25925 |
BoltonBailey author:BoltonBailey |
feat: file for lemmas about MvPolynomials over NoZeroDivisors |
This PR creates a new file for lemmas about `MvPolynomial`s over rings which are `NoZeroDivisors`, to make modified versions of lemmas like `degreeOf_C_mul`.
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
- [x] depends on: #25926 [We need this lemma to establish fact about degreeOf n (p + q)]
|
t-algebra label:t-algebra$ |
85/0 |
Mathlib/Algebra/MvPolynomial/NoZeroDivisors.lean |
1 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
0-50216 13 hours ago |
0-56784 15 hours ago |
0-0 0 seconds |
| 31986 |
SnirBroshi author:SnirBroshi |
feat(Data/List/Cycle): `{next,prev}_getElem` without `Nodup` + infix theorems |
- `List.next`:
- `l.next a = l[l.idxOf a + 1]` and `[a, l.next a] <:+: l`
- unless `a` is the last element, in which case `l.next l.getLast = l.head`
- and in general `l.next a = l[(l.idxOf a + 1) % l.length]`
- `List.prev`:
- `l.prev a = l[l.idxOf a - 1]` and `[l.prev a, a] <:+: l`
- unless `a` is the first element, in which case `l.prev l.head = l.getLast`
- and in general `l.prev a = l[(l.idxOf a + (l.length - 1)) % l.length]`
---
Many of the existing theorems assume `l.Nodup`, so this proves the general case.
[](https://gitpod.io/from-referrer/)
|
t-data
awaiting-author
|
97/0 |
Mathlib/Data/List/Cycle.lean |
1 |
7 |
['Vierkantor', 'github-actions'] |
Vierkantor and pechersky assignee:Vierkantor assignee:pechersky |
0-49859 13 hours ago |
0-49859 13 hours ago |
11-43957 11 days |
| 31689 |
barni120400 author:barni120400 |
feat(Combinatorics/Additive): subset-sum definition and basic properties |
Add subset-sum definition, basic properties and cardinality lower bound |
new-contributor
t-combinatorics
|
139/0 |
Mathlib.lean,Mathlib/Combinatorics/Additive/SubsetSum.lean,docs/references.bib |
3 |
67 |
['Rob23oba', 'YaelDillies', 'barni120400', 'github-actions', 'kckennylau', 'mathlib4-merge-conflict-bot'] |
nobody |
0-49757 13 hours ago |
0-49757 13 hours ago |
0-80376 22 hours |
| 32437 |
WenrongZou author:WenrongZou |
feat(Algebra/Category/ModuleCat/Sheaf/Quasicoherent): construction of `Presentation` |
We construct presentation of sheaf of module by sequence and add `Presentation.map`.
This contribution was created as part of the Heidelberg Lean workshop "Formalising algebraic geometry" in November 2025.
Co-authored-by: William Coram @WilliamCoram
Co-authored-by: Andrew Yang @erdOne
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-algebra
label:t-algebra$ |
90/0 |
Mathlib/Algebra/Category/ModuleCat/Sheaf/Quasicoherent.lean |
1 |
1 |
['github-actions'] |
nobody |
0-48582 13 hours ago |
0-48665 13 hours ago |
0-48710 13 hours |
| 32436 |
thorimur author:thorimur |
feat: `unusedFactInType` linter |
---
[](https://gitpod.io/from-referrer/)
|
t-linter |
55/3 |
Mathlib/Init.lean,Mathlib/Tactic/Linter/UnusedInstancesInType.lean |
2 |
1 |
['github-actions'] |
nobody |
0-44904 12 hours ago |
0-48710 13 hours ago |
0-0 0 seconds |
| 32281 |
ajirving author:ajirving |
feat(NumberTheory.Chebyshev): prove connection between prime counting and theta |
Uses Abel summation to express the prime counting function in terms of the Chebyshev theta function. This upstreams some results from PrimeNumberTheoremAnd.
---
- [ ] depends on: #32247
[](https://gitpod.io/from-referrer/)
|
large-import
new-contributor
t-number-theory
WIP
|
97/0 |
Mathlib/NumberTheory/Chebyshev.lean |
1 |
4 |
['ajirving', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
0-43672 12 hours ago |
0-43680 12 hours ago |
0-1805 30 minutes |
| 31133 |
thorimur author:thorimur |
feat(Linter): combinators for linter option boilerplate |
Provides simple combinators `whenLinterOption` and `whenNotLinterOption` to parallel `whenPPOption` and `whenNotPPOption`, and bundles `withSetOptionIn` and `whenLinterOption` into `whenLinterActivated`.
Currently, a typical linter action uses
```lean
run := withSetOptionIn fun stx => do
unless getLinterValue linter.foo (← getLinterOptions) do
return
...
```
This allows us to simply write
```lean
run := whenLinterActivated linter.foo fun stx => do
...
```
Using these combinators in Mathlib's linters is left to a subsequent PR (#31134).
Since this is a utility used in basic linters, including the header linter, we exclude it from `lint-style`.
---
I'm not sure I'm doing the right thing here re: Mathlib.Init. What exactly should happen?
[](https://gitpod.io/from-referrer/)
|
t-linter
t-meta
|
74/1 |
Mathlib.lean,Mathlib/Lean/Linter.lean,scripts/lint-style.lean |
3 |
11 |
['Vierkantor', 'adomani', 'github-actions', 'mathlib4-merge-conflict-bot', 'thorimur'] |
adomani assignee:adomani |
0-42380 11 hours ago |
0-42846 11 hours ago |
26-48223 26 days |
| 32439 |
joelriou author:joelriou |
feat(Algebra/Homology): morphisms in the derived category between single complexes |
When `Ext` groups of an abelian category are `w`-small, the type of morphisms in the derived category between complexes that are cohomologically in a single degree are also `w`-small.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-category-theory
label:t-algebra$ |
87/0 |
Mathlib.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/Basic.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/TStructure.lean,Mathlib/Algebra/Homology/DerivedCategory/TStructure.lean |
4 |
1 |
['github-actions'] |
nobody |
0-41718 11 hours ago |
0-43243 12 hours ago |
0-43294 12 hours |
| 32363 |
euprunin author:euprunin |
chore: golf using `simpa` |
---
Trace profiling results (shown if ≥10 ms before or after):
* `WeierstrassCurve.Affine.addPolynomial_slope`: 2030 ms before, 1356 ms after 🎉
* `List.Ico.trichotomy`: <10 ms before, 17 ms after
* `List.mk_mem_sym2`: 120 ms before, 90 ms after 🎉
* `Equiv.Perm.set_support_mul_subset`: <10 ms before, 25 ms after
* `Equiv.Perm.support_extend_domain`: 29 ms before, 66 ms after
This golfing PR is batched under the following guidelines:
* Up to 5 changed files per PR
* Up to 25 changed declarations per PR
* Up to 100 changed lines per PR
---
[](https://gitpod.io/from-referrer/)
|
|
6/48 |
Mathlib/AlgebraicGeometry/EllipticCurve/Affine/Formula.lean,Mathlib/Data/Array/Extract.lean,Mathlib/Data/List/Intervals.lean,Mathlib/Data/List/Sym.lean,Mathlib/GroupTheory/Perm/Support.lean |
5 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
0-41243 11 hours ago |
0-41264 11 hours ago |
2-15478 2 days |
| 32320 |
euprunin author:euprunin |
experiment(Algebra): measure the impact of removing redundant tactic invocations (WIP) |
---
**Note: WIP. Do not merge.**
This PR benchmarks the impact of removing tactic invocations that appear to be "technically redundant".
Note: A tactic invocation being technically redundant does not necessarily mean that we want to remove it.
The following tactics were blacklisted and therefore not removed even when they were detected as technically redundant:
* `change`
* `clear`
* `convert`
* `refine`
* `replace`
* `rw`
* `simp_rw`
* `simp`
If you think any tactics should be added to (or removed from) this blacklist, please let me know.
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
WIP
label:t-algebra$ |
1/25 |
Mathlib/Algebra/Algebra/Bilinear.lean,Mathlib/Algebra/BigOperators/Finsupp/Basic.lean,Mathlib/Algebra/BigOperators/Group/Finset/Defs.lean,Mathlib/Algebra/Category/Grp/EpiMono.lean,Mathlib/Algebra/ContinuedFractions/Computation/CorrectnessTerminating.lean,Mathlib/Algebra/ContinuedFractions/Computation/TerminatesIffRat.lean,Mathlib/Algebra/Group/Nat/Range.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/Basic.lean,Mathlib/Algebra/Homology/TotalComplexShift.lean,Mathlib/Algebra/Lie/Weights/RootSystem.lean,Mathlib/Algebra/Module/LinearMap/Polynomial.lean,Mathlib/Algebra/Order/Module/HahnEmbedding.lean,Mathlib/Algebra/Polynomial/Eval/Defs.lean,Mathlib/Algebra/Polynomial/Eval/Irreducible.lean |
14 |
7 |
['euprunin', 'github-actions', 'leanprover-radar', 'mathlib4-merge-conflict-bot'] |
nobody |
0-41190 11 hours ago |
0-41211 11 hours ago |
0-22 22 seconds |
| 31147 |
daefigueroa author:daefigueroa |
feat(Dynamics): point transitive monoid actions and transitive points |
We define point transitivity for a monoid action on a topological space and define the set of transitive points. We add some basic lemmas and implications between topological transitivity and point transitivity.
---
- [x] depends on: #28001
[](https://gitpod.io/from-referrer/) |
new-contributor
t-dynamics
|
114/6 |
Mathlib/Dynamics/Transitive.lean |
1 |
4 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
sgouezel assignee:sgouezel |
0-40082 11 hours ago |
15-86115 15 days ago |
14-66922 14 days |
| 32441 |
euprunin author:euprunin |
chore(Algebra/DirectSum): remove use of `erw` in `mul_eq_dfinsuppSum` |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
2/4 |
Mathlib/Algebra/DirectSum/Ring.lean |
1 |
1 |
['github-actions'] |
nobody |
0-37680 10 hours ago |
0-37691 10 hours ago |
0-37728 10 hours |
| 32442 |
joelriou author:joelriou |
feat(CategoryTheory/Localization): inverse in `SmallShiftedHom` |
The post/precomposition on the types `SmallShiftedHom W` with a morphism which satisfies `W` is a bijection.
---
[](https://gitpod.io/from-referrer/)
|
t-category-theory |
109/0 |
Mathlib/CategoryTheory/Localization/SmallShiftedHom.lean |
1 |
1 |
['github-actions'] |
nobody |
0-36078 10 hours ago |
0-36374 10 hours ago |
0-36352 10 hours |
| 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
---
- [x] depends on: #27520
- [x] depends on: #27538
- [x] depends on: #27510
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
large-import
|
126/3 |
Mathlib/Order/KrullDimension.lean,Mathlib/RingTheory/Ideal/Height.lean,Mathlib/RingTheory/KrullDimension/Polynomial.lean,Mathlib/RingTheory/Localization/AtPrime/Basic.lean,Mathlib/RingTheory/Polynomial/Basic.lean |
5 |
n/a |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
0-35509 9 hours ago |
unknown |
unknown |
| 31034 |
chrisflav author:chrisflav |
feat(RingTheory/Extension/Cotangent): basis of free cotangent space can be realized as a presentation |
Let `S` be a finitely presented `R`-algebra and suppose `P : R[X] → S` generates `S` with
kernel `I`. In this PR we show that if `I/I²` is free, there exists an `R`-presentation `P'` of `S`
extending `P` with kernel `I'`, such that `I'/I'²` is free on the images of the relations of `P'`.
From Pi1.
---
- [x] depends on: #30955
- [x] depends on: #31036
[](https://gitpod.io/from-referrer/)
|
t-ring-theory |
327/0 |
Mathlib.lean,Mathlib/RingTheory/Extension/Cotangent/Basis.lean,Mathlib/RingTheory/Extension/Generators.lean,Mathlib/RingTheory/Extension/Presentation/Basic.lean |
4 |
13 |
['chrisflav', 'erdOne', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
alreadydone assignee:alreadydone |
0-35083 9 hours ago |
0-58646 16 hours ago |
6-43871 6 days |
| 32005 |
metakunt author:metakunt |
feat(Algebra/Polynomial/Basic): Add ofMultiset |
Add Polynomial.ofMultiset to eventually refactor theorems using Multiset.map.prod paradigm in future PR's.
Discussion: https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Adding.20Polynomial.2EfromRoots.3F/with/558903708
|
new-contributor
t-algebra
label:t-algebra$ |
80/55 |
Mathlib/Algebra/Polynomial/Basic.lean,Mathlib/Algebra/Polynomial/BigOperators.lean,Mathlib/Algebra/Polynomial/Factors.lean,Mathlib/Algebra/Polynomial/Roots.lean,Mathlib/Algebra/Polynomial/Splits.lean,Mathlib/Analysis/Normed/Unbundled/SpectralNorm.lean,Mathlib/FieldTheory/IsAlgClosed/AlgebraicClosure.lean,Mathlib/FieldTheory/IsAlgClosed/Basic.lean,Mathlib/FieldTheory/KummerExtension.lean,Mathlib/FieldTheory/Minpoly/ConjRootClass.lean,Mathlib/FieldTheory/SeparableDegree.lean,Mathlib/RingTheory/Polynomial/Cyclotomic/Basic.lean,Mathlib/RingTheory/Polynomial/IsIntegral.lean,Mathlib/RingTheory/Polynomial/Vieta.lean |
14 |
11 |
['github-actions', 'mathlib4-merge-conflict-bot', 'metakunt', 'ocfnash'] |
ocfnash assignee:ocfnash |
0-31763 8 hours ago |
0-31763 8 hours ago |
5-33482 5 days |
| 32379 |
marwahaha author:marwahaha |
feat(Analysis/SpecialFunctions): prove expNegInvGlue is not analytic at zero |
Previously expNegInvGlue was shown to have a property not possible by analytic functions; here we add a proof that the function is not analytic.
Closes #31209
---
(this question was answered below) I don't understand, which will become the commit message? Is it the text above the `---` in this textbox? Or the title of the Github PR? To be safe I did not include any text above the `---`. I found the examples in https://leanprover-community.github.io/contribute/commit.html conflicting with itself, and the text in the GitHub PR template.
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-analysis
|
10/0 |
Mathlib/Analysis/SpecialFunctions/SmoothTransition.lean |
1 |
28 |
['LLaurance', 'adomani', 'b-mehta', 'github-actions', 'j-loreaux', 'marwahaha', 'mcdoll'] |
nobody |
0-31640 8 hours ago |
0-33157 9 hours ago |
2-7761 2 days |
| 31406 |
JovanGerb author:JovanGerb |
feat(push_neg): `push_neg +distrib` syntax |
This PR adds the syntax `push_neg +distrib`, `by_cases! +distrib`, `contrapose! +distrib` and `by_contra! +distrib`. This is much more convenient to use than writing out `set_option push_neg.use_distrib true in`. All uses of the `set_option` version have been replaced with the new syntax.
I also add a missing `namespace` in the definition of `by_cases!` and `by_contra!`
---
- [x] depends on: #31510
- [x] depends on: #32230
[](https://gitpod.io/from-referrer/)
|
t-meta
awaiting-author
|
132/67 |
Mathlib/Algebra/Group/Pointwise/Finset/Basic.lean,Mathlib/Algebra/Group/Pointwise/Set/Basic.lean,Mathlib/Algebra/Group/UniqueProds/Basic.lean,Mathlib/Analysis/SpecialFunctions/BinaryEntropy.lean,Mathlib/Data/EReal/Operations.lean,Mathlib/Data/Finite/Prod.lean,Mathlib/Geometry/Euclidean/Angle/Oriented/Basic.lean,Mathlib/LinearAlgebra/LinearIndependent/Defs.lean,Mathlib/NumberTheory/Padics/PadicVal/Basic.lean,Mathlib/NumberTheory/WellApproximable.lean,Mathlib/Order/LiminfLimsup.lean,Mathlib/Order/Quotient.lean,Mathlib/RingTheory/Ideal/Basic.lean,Mathlib/SetTheory/Cardinal/Arithmetic.lean,Mathlib/Tactic/ByCases.lean,Mathlib/Tactic/ByContra.lean,Mathlib/Tactic/Contrapose.lean,Mathlib/Tactic/Push.lean,MathlibTest/Contrapose.lean,MathlibTest/byContra.lean,MathlibTest/push_neg.lean |
21 |
25 |
['JovanGerb', 'Vierkantor', 'github-actions', 'grunweg', 'leanprover-bot', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
grunweg assignee:grunweg |
0-30241 8 hours ago |
3-32019 3 days ago |
12-8361 12 days |
| 30853 |
JovanGerb author:JovanGerb |
feat(LinearAlgebra/AffineSpace/Simplex): `CoeFun` instance for `Simplex` |
This PR introduces the notation `s i` to refer to the `i`th vertex of simplex `s`, which replaces the current `s.points i`. It does this by adding a `CoeFun` instance.
I first tried using `FunLike`, but this came with some different problems related to discrimination tree indexing in `simp`.
---
[](https://gitpod.io/from-referrer/)
|
|
381/371 |
Archive/Imo/Imo2019Q2.lean,Mathlib/Analysis/Convex/Between.lean,Mathlib/Analysis/Normed/Affine/Simplex.lean,Mathlib/Geometry/Euclidean/Altitude.lean,Mathlib/Geometry/Euclidean/Angle/Sphere.lean,Mathlib/Geometry/Euclidean/Circumcenter.lean,Mathlib/Geometry/Euclidean/Incenter.lean,Mathlib/Geometry/Euclidean/MongePoint.lean,Mathlib/Geometry/Euclidean/Projection.lean,Mathlib/Geometry/Euclidean/SignedDist.lean,Mathlib/Geometry/Euclidean/Simplex.lean,Mathlib/LinearAlgebra/AffineSpace/FiniteDimensional.lean,Mathlib/LinearAlgebra/AffineSpace/Simplex/Basic.lean,Mathlib/LinearAlgebra/AffineSpace/Simplex/Centroid.lean,scripts/nolints.json |
15 |
11 |
['JovanGerb', 'github-actions', 'jsm28', 'mathlib4-merge-conflict-bot'] |
mattrobball assignee:mattrobball |
0-29861 8 hours ago |
0-29878 8 hours ago |
40-81032 40 days |
| 32414 |
SnirBroshi author:SnirBroshi |
feat(NumberTheory/ArithmeticFunction/Carmichael): Carmichael totient function |
Define `ArithmeticFunction.Carmichael`, the Carmichael function `λ`, also known as the reduced totient function.
Prove the known formula for `λ n` in terms of the prime factorization of `n`, along with some useful properties:
- `a ^ λ n = 1`
- `λ n ∣ φ n`
- `a ∣ b → λ a ∣ λ b`
- `λ (lcm a b) = lcm (λ a) (λ b)`
---
I'm open to suggestions on where to place the `Finset.lcm` lemmas, I created a separate file to avoid adding imports to existing files.
I'm also wondering whether to change the `HasEnoughRootsOfUnity` here to use `Carmichael`: https://github.com/leanprover-community/mathlib4/blob/6a7385f3f6d2c0b674e3ecd96506e57737b77064/Mathlib/NumberTheory/DirichletCharacter/Orthogonality.lean#L31
[](https://gitpod.io/from-referrer/)
|
|
211/0 |
Mathlib.lean,Mathlib/Algebra/GCDMonoid/FinsetLemmas.lean,Mathlib/NumberTheory/ArithmeticFunction/Carmichael.lean |
3 |
1 |
['github-actions'] |
nobody |
0-29859 8 hours ago |
1-19878 1 day ago |
1-19855 1 day |
| 32176 |
JovanGerb author:JovanGerb |
feat(translate): refactor `applyReplacementFun` and more |
This PR cleans up a lot of the `to_additive` implementation.
`applyReplacementFun` is cleaned up:
- Instead of running `shouldTranslate` at every single constant appliaction, we now only run it on constant applications where the head constant can actually be translated
- The option for translating numerals was mistakenly not actually looked at. This means that `to_dual` would translate the numeral 1 to 0. This is fixed.
- We remove the `Expr.proj` handling, because these are already handled by `expand`.
- The `if gf.isBVar && x.isLit` is now not needed anymore and is removed.
- It now uses `memoFix` instead of `Lean.Expr.replaceRec`, which will is more transparent, and will allow us to change the monad in the future if needed.
Some more cleanups:
- `transformDecl` has been removed/inlined since it is a small function only used once.
- `transformDeclAux` has been renamed to `transformDeclRec` (as it recursively transforms the declarations appearing inside the declaration). It now recursively calls itself with an empty `reorder` and `dontTranslate`, which helps avoid a case split.
- In `ToAdditive` and `ToDual`, an unused piece of syntax has been removed.
- `memoFix` has been reimplemented to actually use pointer equality.
---
[](https://gitpod.io/from-referrer/)
|
t-meta |
79/132 |
Mathlib/Tactic/Translate/Core.lean,Mathlib/Tactic/Translate/ToAdditive.lean,Mathlib/Tactic/Translate/ToDual.lean,Mathlib/Util/MemoFix.lean,MathlibTest/ToDual.lean,MathlibTest/toAdditive.lean |
6 |
13 |
['JovanGerb', 'github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'leanprover-radar', 'mathlib4-merge-conflict-bot'] |
bryangingechen assignee:bryangingechen |
0-29705 8 hours ago |
0-29724 8 hours ago |
6-86185 6 days |
| 31803 |
grunweg author:grunweg |
chore(Tactic/Linters): remove `public section` |
Mostly as a learning exercise for me to understand the module system better.
---
- [x] depends on: #31823 (to make visibility changes just for tests a conscious choice)
[](https://gitpod.io/from-referrer/)
|
t-linter |
119/101 |
Mathlib/Tactic/Linter/CommandRanges.lean,Mathlib/Tactic/Linter/CommandStart.lean,Mathlib/Tactic/Linter/DeprecatedModule.lean,Mathlib/Tactic/Linter/DeprecatedSyntaxLinter.lean,Mathlib/Tactic/Linter/DirectoryDependency.lean,Mathlib/Tactic/Linter/DocPrime.lean,Mathlib/Tactic/Linter/DocString.lean,Mathlib/Tactic/Linter/FindDeprecations.lean,Mathlib/Tactic/Linter/FlexibleLinter.lean,Mathlib/Tactic/Linter/GlobalAttributeIn.lean,Mathlib/Tactic/Linter/HashCommandLinter.lean,Mathlib/Tactic/Linter/HaveLetLinter.lean,Mathlib/Tactic/Linter/Header.lean,Mathlib/Tactic/Linter/Lint.lean,Mathlib/Tactic/Linter/MinImports.lean,Mathlib/Tactic/Linter/Multigoal.lean,Mathlib/Tactic/Linter/OldObtain.lean,Mathlib/Tactic/Linter/PPRoundtrip.lean,Mathlib/Tactic/Linter/Style.lean,Mathlib/Tactic/Linter/TextBased.lean,Mathlib/Tactic/Linter/UnusedTactic.lean,Mathlib/Tactic/Linter/UnusedTacticExtension.lean,Mathlib/Tactic/Linter/UpstreamableDecl.lean,MathlibTest/CommandStart.lean,MathlibTest/FlexibleLinter.lean,MathlibTest/ForbiddenModuleNames.lean,MathlibTest/ModuleCasing.lean |
27 |
28 |
['JovanGerb', 'Vierkantor', 'github-actions', 'grunweg', 'leanprover-bot', 'leanprover-radar', 'mathlib4-dependent-issues-bot'] |
thorimur assignee:thorimur |
0-29229 8 hours ago |
0-29346 8 hours ago |
15-18837 15 days |
| 32403 |
FLDutchmann author:FLDutchmann |
fix(FieldSimp): `declaration has free variables` kernel errors |
Fix a bug in `field_simp` that produces a `(kernel) declaration has free variables '_example'` error which was caused by a misconfigured `simp` call.
---
The first new test produces this error on the current version of mathlib. What I believe is happening is that the discharger is using the `x != 0` hypothesis in the `then` branch, at which point that result is cached by `simp` and used in the `else` branch.
```
import Mathlib
/- (kernel) declaration has free variables '_example' -/
example {x y : ℚ}: (if x ≠ 0 then x / x else x / x) = 1 := by
field_simp
/- ⊢ (if x ≠ 0 then 1 else 1) = 1 -/
sorry
```
Edit: As @__JovanGerb__ pointed out, the correct solution was to set the `wellBehavedDischarge` flag to false, so that `simp` clears the cache more agressively. We might also want to turn on `contextual` in the future, but this would change the behaviour of `field_simp` by adding additional lemmas to the simp context. For now I propose a fix with a minimal change in behaviour.
Marking the simp context that calls the discharger as contextual appears to fix the issue, presumably by more aggressively pruning the cache. What I don't understand at this point, is why the discharger ever even had access to that hypothesis, given that contextual was set to false.
cc @JovanGerb : You understand the simp cache much better than I. Is there another bug here that I'm missing?
[](https://gitpod.io/from-referrer/)
|
t-meta |
53/6 |
Mathlib/Tactic/Abel.lean,Mathlib/Tactic/FieldSimp.lean,Mathlib/Tactic/Ring/RingNF.lean,Mathlib/Util/AtomM/Recurse.lean,MathlibTest/FieldSimp.lean |
5 |
4 |
['FLDutchmann', 'JovanGerb', 'github-actions', 'leanprover-radar'] |
nobody |
0-29223 8 hours ago |
0-62928 17 hours ago |
1-57034 1 day |
| 32340 |
SnirBroshi author:SnirBroshi |
doc(1000.yaml): add `ZMod` version of Chinese remainder theorem |
The `Ideal` statement is from leanprover-community/mathlib3#774 and the `ZMod` statement is from leanprover-community/mathlib3#8356.
---
There are many other versions of CRT in Mathlib:
- [`Mathlib.Data.Nat.ChineseRemainder`](https://leanprover-community.github.io/mathlib4_docs/Mathlib/Data/Nat/ChineseRemainder.html)
- [`Nat.modEq_and_modEq_iff_modEq_mul`](https://leanprover-community.github.io/mathlib4_docs/Mathlib/Data/Nat/ModEq.html#Nat.modEq_and_modEq_iff_modEq_mul)
- [`ZMod.prodEquivPi`](https://leanprover-community.github.io/mathlib4_docs/Mathlib/Data/ZMod/QuotientRing.html#ZMod.prodEquivPi)
- [`ZMod.equivPi`](https://leanprover-community.github.io/mathlib4_docs/Mathlib/Data/ZMod/QuotientRing.html#ZMod.equivPi)
- [`IsDedekindDomain.quotientEquivPiOfProdEq`](https://leanprover-community.github.io/mathlib4_docs/Mathlib/RingTheory/DedekindDomain/Ideal/Lemmas.html#IsDedekindDomain.quotientEquivPiOfProdEq)
- [`IsDedekindDomain.quotientEquivPiFactors`](https://leanprover-community.github.io/mathlib4_docs/Mathlib/RingTheory/DedekindDomain/Ideal/Lemmas.html#IsDedekindDomain.quotientEquivPiFactors)
- [`IsDedekindDomain.quotientEquivPiOfFinsetProdEq`](https://leanprover-community.github.io/mathlib4_docs/Mathlib/RingTheory/DedekindDomain/Ideal/Lemmas.html#IsDedekindDomain.quotientEquivPiOfFinsetProdEq)
- [`Mathlib.RingTheory.Ideal.Quotient.ChineseRemainder`](https://leanprover-community.github.io/mathlib4_docs/Mathlib/RingTheory/Ideal/Quotient/ChineseRemainder.html)
But I think at least one statement about `Nat` or `ZMod` should be listed under CRT in the 1000 list, next to the algebraic version.
[](https://gitpod.io/from-referrer/)
|
|
5/1 |
docs/1000.yaml |
1 |
2 |
['github-actions'] |
nobody |
0-29139 8 hours ago |
3-16346 3 days ago |
3-16323 3 days |
| 32416 |
kim-em author:kim-em |
feat(TacticAnalysis): add generic env var-based tryAtEachStep linter |
## Summary
Adds a generic `tryAtEachStepFromEnv` tactic analysis linter that reads the tactic to try from environment variables. This allows hammer-bench and similar tools to test arbitrary tactics without requiring Mathlib code changes.
- `TRY_AT_EACH_STEP_TACTIC`: The tactic syntax to try (e.g., "grind +suggestions")
- `TRY_AT_EACH_STEP_LABEL`: Human-readable label for output (optional)
Uses `captureException` with `tacticSeq.fn` to parse tactic strings, following Kenny Lau's suggestion from [Zulip](https://leanprover.zulipchat.com/#narrow/channel/113488-general/topic/piggy.20back.20off.20of.20the.20lean4.20parser). This enables support for tactic sequences like "simp; grind".
Also removes the unnecessary `Mathlib.Init` import from `ParseCommand.lean` to avoid import cycles.
🤖 Prepared with Claude Code |
large-import |
221/8 |
Mathlib/Init.lean,Mathlib/Tactic/TacticAnalysis/Declarations.lean,Mathlib/Util/ParseCommand.lean,MathlibTest/TacticAnalysis.lean,MathlibTest/tryAtEachStep.lean |
5 |
10 |
['dwrensha', 'github-actions', 'grunweg', 'kim-em'] |
nobody |
0-28681 7 hours ago |
0-82020 22 hours ago |
1-3507 1 day |
| 32445 |
vihdzp author:vihdzp |
chore: avoid non-terminal simp |
---
There's six instances of `-Function.iterate_succ` in Mathlib besides this, perhaps someone should look into that?
[](https://gitpod.io/from-referrer/)
|
t-order
easy
|
2/5 |
Mathlib/Order/Iterate.lean |
1 |
1 |
['github-actions'] |
nobody |
0-28339 7 hours ago |
0-28438 7 hours ago |
0-28478 7 hours |
| 31886 |
CoolRmal author:CoolRmal |
feat: the family of limits in probability of sequences of uniformly integrable random variables is uniformly integrable |
---
[](https://gitpod.io/from-referrer/)
|
brownian
t-measure-probability
|
73/9 |
Mathlib/MeasureTheory/Function/ConvergenceInMeasure.lean,Mathlib/MeasureTheory/Function/UniformIntegrable.lean |
2 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
EtienneC30 assignee:EtienneC30 |
0-27434 7 hours ago |
0-72540 20 hours ago |
0-74138 20 hours |
| 30241 |
joelriou author:joelriou |
feat(CategoryTheory): locally presentable categories and strong generators |
Let `C` be category that is locally `w`-small and has colimits of shape `w`. Then, `C` is locally `κ`-presentable iff it has a strong generator consisting of `κ`-presentable objects.
(This is a draft.)
---
- [ ] depends on: #30459
- [ ] depends on: #30168
- [ ] depends on: #29565
- [x] depends on: #30269
- [x] depends on: #29851
- [x] depends on: #29881
- [x] depends on: #29903
- [x] depends on: #29854
- [x] depends on: #30160
- [x] depends on: #29556
- [x] depends on: #29519
- [x] depends on: #29518
- [x] depends on: #29543
[](https://gitpod.io/from-referrer/)
|
t-category-theory |
774/87 |
Mathlib.lean,Mathlib/CategoryTheory/EssentiallySmall.lean,Mathlib/CategoryTheory/Functor/KanExtension/Dense.lean,Mathlib/CategoryTheory/Generator/Basic.lean,Mathlib/CategoryTheory/Limits/HasLimits.lean,Mathlib/CategoryTheory/ObjectProperty/Basic.lean,Mathlib/CategoryTheory/ObjectProperty/ClosedUnderIsomorphisms.lean,Mathlib/CategoryTheory/ObjectProperty/ColimitsCardinalClosure.lean,Mathlib/CategoryTheory/ObjectProperty/ColimitsOfShape.lean,Mathlib/CategoryTheory/ObjectProperty/CompleteLattice.lean,Mathlib/CategoryTheory/ObjectProperty/Equivalence.lean,Mathlib/CategoryTheory/ObjectProperty/Small.lean,Mathlib/CategoryTheory/Presentable/Basic.lean,Mathlib/CategoryTheory/Presentable/CardinalFilteredPresentation.lean,Mathlib/CategoryTheory/Presentable/Limits.lean,Mathlib/CategoryTheory/Presentable/LocallyPresentable.lean,Mathlib/CategoryTheory/Presentable/StrongGenerator.lean,Mathlib/CategoryTheory/SmallRepresentatives.lean |
18 |
5 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
0-26008 7 hours ago |
26-39964 26 days ago |
0-1 1 second |
| 31174 |
joelriou author:joelriou |
refactor(AlgebraicTopology): refactor the homotopy category and the nerve adjunction |
This PR completely refactors the adjunction between quivers and reflexive quivers, the homotopy category of a simplicial set, and the adjunction between (2-truncated) simplicial sets and `Cat` (which involves the homotopy category of a simplicial set and the nerve of a category).
The general principle which is applied here is that for any (strictly functorial) construction involving quivers, refl. quivers or categories, the constructions and the basic API are first done in the unbundled setting (a type with a `Category/Quiver/...` instance), and only at the very end, the functors involving `Cat/Quiv/...` and the adjunctions are defined in the bundled situation. This gives cleaner code and improves automation.
The adjunctions are now constructed by defining the `homEquiv` rather than by constructing the unit/counit. This emphasizes a little bit more the universal properties of the constructions. The unit/counit can be recovered from the `homEquiv` (and it seems they are definitionally to the previous definitions).
---
- [x] depends on: #31248
- [x] depends on: #31250
- [x] depends on: #31254
- [x] depends on: #31274
- [x] depends on: #31265
[](https://gitpod.io/from-referrer/)
|
t-algebraic-topology |
970/736 |
Mathlib/AlgebraicTopology/SimplicialSet/CompStruct.lean,Mathlib/AlgebraicTopology/SimplicialSet/HomotopyCat.lean,Mathlib/AlgebraicTopology/SimplicialSet/Nerve.lean,Mathlib/AlgebraicTopology/SimplicialSet/NerveAdjunction.lean,Mathlib/AlgebraicTopology/SimplicialSet/Path.lean,Mathlib/CategoryTheory/Category/ReflQuiv.lean,Mathlib/CategoryTheory/Monoidal/Closed/Cartesian.lean,Mathlib/CategoryTheory/MorphismProperty/Basic.lean,Mathlib/CategoryTheory/MorphismProperty/Composition.lean,Mathlib/CategoryTheory/PathCategory/Basic.lean,Mathlib/Combinatorics/Quiver/ReflQuiver.lean |
11 |
32 |
['github-actions', 'joelriou', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'robin-carlier'] |
nobody |
0-26006 7 hours ago |
4-8012 4 days ago |
4-83362 4 days |
| 31452 |
jsm28 author:jsm28 |
feat(Analysis/Convex/StrictCombination): convex combinations in strictly convex sets and spaces |
Add various lemmas that combinations of points (nonnegative weights, at least two weights of distinct points nonzero) in strictly convex sets lie in the interior of that set, or in strictly convex spaces or affine spaces for such spaces lie in a ball when the points lie in the corresponding closed ball.
These are analogous to existing lemmas for convex combinations and for pairs of points in strictly convex sets or spaces. In particular, the way `StrictConvex.centerMass_mem_interior` is stated with various hypotheses after the colon follows how `Convex.centerMass_mem` is stated (the hypotheses could of course move before the colon if they were then generalized for the induction).
Convenience lemmas for the cases of `closedInterior` (excluding vertices) of a simplex, and `interior` of a simplex, are included. https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Triangle.20interior.20and.20its.20circumsphere/with/540305703 requested such a statement (in a different form). They don't include anything for bundled spheres since those are currently defined in `Mathlib.Geometry.Euclidean`, though given a suitable more generic name for the bundled sphere structure, various basic material about such spheres could move to a more generic metric space location, at which point it would be reasonable to add versions of these statements that use bundled spheres.
---
- [ ] depends on: #31450
- [ ] depends on: #31451
[](https://gitpod.io/from-referrer/)
|
t-convex-geometry |
165/0 |
Mathlib.lean,Mathlib/Analysis/Convex/StrictCombination.lean |
2 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
YaelDillies assignee:YaelDillies |
0-26005 7 hours ago |
15-76570 15 days ago |
20-63803 20 days |
| 31757 |
mcdoll author:mcdoll |
feat(Analysis/Distribution): definition of tempered distributions |
Define the space of tempered distributions as an abbreviation. We also prove the abstract convergence results
for `PointwiseConvergenceCLM` and define the Fourier transform on tempered distributions.
There is a bit of disagreement in the literature about which is the correct topology on tempered distributions. For practical reasons, we will use the pointwise topology, but we might switch later to the bounded topology, if the abstract functional analysis is developed enough to prove the same statements.
---
- [x] depends on: #31756
- [x] depends on: #31577
- [x] depends on: #31760
[](https://gitpod.io/from-referrer/)
|
t-analysis |
225/9 |
Mathlib.lean,Mathlib/Analysis/Distribution/TemperedDistribution.lean,Mathlib/Analysis/LocallyConvex/PointwiseConvergence.lean,Mathlib/Topology/Algebra/Module/PointwiseConvergence.lean,docs/overview.yaml,docs/undergrad.yaml |
6 |
6 |
['ADedecker', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'mcdoll'] |
nobody |
0-26004 7 hours ago |
3-28104 3 days ago |
3-28089 3 days |
| 32079 |
wwylele author:wwylele |
feat(Topology): UniformContinuous version of uniform limit theorem |
Upgrade the following theorems to UniformContinuous
- `continuousOn_of_uniform_approx_of_continuousOn` -> `uniformContinuousOn_of_uniform_approx_of_uniformContinuousOn`
- `continuous_of_uniform_approx_of_continuous` -> `uniformContinuous_of_uniform_approx_of_uniformContinuous`
- `TendstoUniformlyOn.continuousOn` -> `TendstoUniformlyOn.uniformContinuousOn`
- `TendstoUniformly.continuous` -> `TendstoUniformly.uniformContinuous`
Co-authored-by: Aaron Liu
---
[](https://gitpod.io/from-referrer/)
|
t-topology |
46/0 |
Mathlib/Topology/UniformSpace/UniformApproximation.lean |
1 |
1 |
['github-actions'] |
nobody |
0-26003 7 hours ago |
10-25131 10 days ago |
10-25173 10 days |
| 32080 |
plp127 author:plp127 |
feat(Topology): Completely Regular Space iff Uniformizable |
This PR continues the work from #24096.
Original PR: https://github.com/leanprover-community/mathlib4/pull/24096
---------
- [x] depends on: #32140 |
t-topology |
137/0 |
Mathlib.lean,Mathlib/Data/Rel.lean,Mathlib/Topology/UniformSpace/Uniformizable.lean |
3 |
3 |
['github-actions', 'grunweg', 'mathlib4-dependent-issues-bot'] |
urkud assignee:urkud |
0-26002 7 hours ago |
7-28982 7 days ago |
8-70466 8 days |
| 32144 |
EtienneC30 author:EtienneC30 |
feat: add a predicate HasGaussianLaw |
Define a predicate `HasGaussianLaw X P`, which states that under the measure `P`, the random variable `X` has a Gaussian distribution, i.e. `IsGaussian (P.map X)`.
---
- [x] depends on: #32280
[](https://gitpod.io/from-referrer/)
|
brownian
t-measure-probability
|
267/0 |
Mathlib.lean,Mathlib/Probability/Distributions/Gaussian/HasGaussianLaw/Basic.lean,Mathlib/Probability/Distributions/Gaussian/HasGaussianLaw/Def.lean |
3 |
4 |
['EtienneC30', 'github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
0-26001 7 hours ago |
3-79856 3 days ago |
7-79316 7 days |
| 32231 |
grunweg author:grunweg |
chore: use the to_fun attribute |
Reduce code duplication using the to_fun attribute.
This is not exhaustive, neither does it constitute an endorsement "we always want to generate the applied form of a lemma".
---
This may also want to wait until copying doc-strings is supported (to avoid regressions on that front),
and until the generated declaration is hoverable (for easier migration to the attribute).
- [x] depends on: #31872
[](https://gitpod.io/from-referrer/)
|
|
74/242 |
Mathlib/Analysis/Analytic/Constructions.lean,Mathlib/Analysis/Meromorphic/Basic.lean |
2 |
6 |
['JovanGerb', 'github-actions', 'grunweg', 'mathlib4-dependent-issues-bot'] |
joneugster assignee:joneugster |
0-26000 7 hours ago |
3-47869 3 days ago |
3-51278 3 days |
| 32297 |
mcdoll author:mcdoll |
feat(Analysis/Distribution): composition of temperate growth functions |
Proves that the composition of temperate growth functions is again of temperate growth. We have to use the explicit bounds, because we want to have the case that the outer function `g` is only temperate on the image of the inner function `f`, to be able to apply this result for `f x = 1 + |x|^2` and `g x = x ^ r` for any real `r`.
---
[](https://gitpod.io/from-referrer/)
|
t-analysis |
91/1 |
Mathlib/Analysis/Distribution/SchwartzSpace.lean,Mathlib/Analysis/Distribution/TemperateGrowth.lean |
2 |
1 |
['github-actions'] |
nobody |
0-25998 7 hours ago |
3-65778 3 days ago |
3-72527 3 days |
| 32303 |
joelriou author:joelriou |
feat(CategoryTheory): commutation of bifunctors to shifts in two variables |
This will be used when formalising triangulated bifunctors.
---
[](https://gitpod.io/from-referrer/)
|
t-category-theory |
148/1 |
Mathlib.lean,Mathlib/CategoryTheory/Center/NegOnePow.lean,Mathlib/CategoryTheory/Shift/CommShiftTwo.lean,Mathlib/CategoryTheory/Shift/Twist.lean |
4 |
1 |
['github-actions'] |
kim-em assignee:kim-em |
0-25997 7 hours ago |
3-60239 3 days ago |
3-71255 3 days |
| 32306 |
plp127 author:plp127 |
fix(depRewrite): make `rw!` cleanup casts correctly |
The tactic `rw!` runs a round of `dsimp` with a minimal configuration, intended to cleanup casts. This minimal configuration is not always enough to fully reduce the casts, and may have other side effects. This PR reimplements the cast cleanup in a way not involving `dsimp` that will fully reduce casts introduced by depRewrite and will not touch other parts of the expression.
---
[](https://gitpod.io/from-referrer/)
|
t-meta |
140/51 |
Mathlib/Tactic/DepRewrite.lean,MathlibTest/depRewrite.lean |
2 |
1 |
['github-actions'] |
adamtopaz assignee:adamtopaz |
0-25996 7 hours ago |
3-67934 3 days ago |
3-67922 3 days |
| 32326 |
chrisflav author:chrisflav |
feat(Algebra/ModuleCat): extension of scalars is comonadic for a faithfully flat algebra |
This is also known as faithfully flat descent, but the proof that these statements indeed imply each other is much longer than this PR (see #24434).
Co-authored-by: Dagur Asgeirsson
Co-authored-by: Jack McKoen
Co-authored-by: Joël Riou
Co-authored-by: Adam Topaz
This contribution was created as part of the AIM workshop
"Formalizing algebraic geometry" in June 2024.
---
This PR continues the work from #14203.
[](https://gitpod.io/from-referrer/)
|
t-ring-theory |
98/0 |
Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/ChangeOfRings.lean,Mathlib/Algebra/Category/ModuleCat/Descent.lean,Mathlib/Algebra/Homology/ShortComplex/ExactFunctor.lean,Mathlib/RingTheory/Flat/FaithfullyFlat/Basic.lean |
5 |
1 |
['github-actions'] |
nobody |
0-25995 7 hours ago |
3-47393 3 days ago |
3-47371 3 days |
| 32444 |
vihdzp author:vihdzp |
feat: `SignType` is a complete linear order |
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-data
t-order
easy
|
3/0 |
Mathlib/Data/Sign/Basic.lean |
1 |
2 |
['github-actions', 'vihdzp'] |
nobody |
0-25664 7 hours ago |
0-25664 7 hours ago |
0-34317 9 hours |
| 32438 |
JovanGerb author:JovanGerb |
feat: unfold-boundaries in `to_dual` |
This PR introduces a new feature to `to_dual` that allows us to have definitions whose dual is not definitionally equal to the dual of the value. This is crucial for many definitions that are dual to something morally but not definitionally. For example, `DecidableLE`, `Set.Ioo`, `Set.Ico`, `CovBy` , `Monotone`.
---
[](https://gitpod.io/from-referrer/)
|
large-import |
285/24 |
Mathlib.lean,Mathlib/Order/Basic.lean,Mathlib/Order/Cover.lean,Mathlib/Order/Defs/LinearOrder.lean,Mathlib/Order/Defs/PartialOrder.lean,Mathlib/Order/Interval/Set/Defs.lean,Mathlib/Tactic.lean,Mathlib/Tactic/ToDual.lean,Mathlib/Tactic/Translate/Core.lean,Mathlib/Tactic/Translate/ToDual.lean,Mathlib/Tactic/Translate/UnfoldBoundary.lean |
11 |
1 |
['github-actions'] |
nobody |
0-25561 7 hours ago |
0-46686 12 hours ago |
0-0 0 seconds |
| 29437 |
SnirBroshi author:SnirBroshi |
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/)
|
t-data
new-contributor
|
102/0 |
Mathlib/Data/Int/Init.lean,Mathlib/Data/Nat/Init.lean,Mathlib/Data/Seq/Basic.lean,Mathlib/Data/Seq/Defs.lean |
4 |
9 |
['SnirBroshi', 'github-actions', 'jcommelin', 'kim-em', 'mathlib4-merge-conflict-bot'] |
pechersky assignee:pechersky |
0-25072 6 hours ago |
0-25072 6 hours ago |
83-32700 83 days |
| 29596 |
alreadydone author:alreadydone |
chore(Algebra): extract `Submonoid.IsLocalizationMap` |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
299/126 |
Mathlib.lean,Mathlib/Algebra/Module/FinitePresentation.lean,Mathlib/GroupTheory/MonoidLocalization/Basic.lean,Mathlib/GroupTheory/MonoidLocalization/Lemmas.lean,Mathlib/GroupTheory/MonoidLocalization/MonoidWithZero.lean,Mathlib/RingTheory/Extension/Presentation/Submersive.lean,Mathlib/RingTheory/Localization/Defs.lean,Mathlib/RingTheory/Localization/FractionRing.lean |
8 |
61 |
['Garmelon', 'alreadydone', 'github-actions', 'jcommelin', 'kckennylau', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'leanprover-radar', 'mathlib4-merge-conflict-bot'] |
kim-em assignee:kim-em |
0-24930 6 hours ago |
1-59078 1 day ago |
74-33193 74 days |
| 32377 |
JovanGerb author:JovanGerb |
chore(Order/BoundedOrder/Basic): use `to_dual` |
Notes:
- `eq_bot_of_minimal` didn't have a dual version, and was unused, so I deprecated it.
- I removed the two >6 month old deprecations.
- The choice of whether to write down top/bot lemmas is mostly based on whichever one came first originally.
---
[](https://gitpod.io/from-referrer/)
|
|
86/235 |
Mathlib/Order/BoundedOrder/Basic.lean,Mathlib/Order/KrullDimension.lean |
2 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
0-23633 6 hours ago |
0-29918 8 hours ago |
1-62381 1 day |
| 32448 |
vihdzp author:vihdzp |
chore(Order/SuccPred/Basic): use `where` notation |
---
[](https://gitpod.io/from-referrer/)
|
t-order
easy
|
20/24 |
Mathlib/Order/SuccPred/Basic.lean |
1 |
1 |
['github-actions'] |
nobody |
0-23154 6 hours ago |
0-23201 6 hours ago |
0-23198 6 hours |
| 32262 |
alreadydone author:alreadydone |
feat(Algebra): Dedekind-finite and stably finite rings |
+ Introduce `IsDedekindFiniteMonoid` and `IsStablyFiniteRing`.
+ Prove equivalent characterizations of Dedekind-finite monoids.
+ Show commutative monoids are Dedekind-finite, and finite monoids/rings are Dedekind-finite/stably-finite. Show Artinian semirings are Dedekind-finite.
+ Show Dedekind-finiteness and stable finiteness are left-right symmetric.
+ Prove matrix characterizations of rank condition and invariant basis number; as consequences, show both properties are left-right symmetric.
+ Show stable finiteness implies the rank condition, generalizing [rankCondition_of_nontrivial_of_commSemiring](https://leanprover-community.github.io/mathlib4_docs/Mathlib/LinearAlgebra/Matrix/InvariantBasisNumber.html#rankCondition_of_nontrivial_of_commSemiring).
+ Reformulate a lemma as saying division rings are stably finite.
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
t-algebra
label:t-algebra$ |
412/76 |
Mathlib.lean,Mathlib/Algebra/Group/Basic.lean,Mathlib/Algebra/Group/Defs.lean,Mathlib/Algebra/Group/Equiv/Defs.lean,Mathlib/Algebra/Group/Hom/Defs.lean,Mathlib/Algebra/Group/Opposite.lean,Mathlib/Algebra/Group/Submonoid/Defs.lean,Mathlib/Algebra/Group/Units/Defs.lean,Mathlib/Algebra/Regular/Basic.lean,Mathlib/Algebra/Ring/Regular.lean,Mathlib/Data/Matrix/Basic.lean,Mathlib/Data/Matrix/Composition.lean,Mathlib/Data/Matrix/Mul.lean,Mathlib/GroupTheory/Finite.lean,Mathlib/LinearAlgebra/FiniteDimensional/Basic.lean,Mathlib/LinearAlgebra/InvariantBasisNumber.lean,Mathlib/LinearAlgebra/Matrix/InvariantBasisNumber.lean,Mathlib/LinearAlgebra/Matrix/SemiringInverse.lean,Mathlib/LinearAlgebra/Matrix/ToLin.lean,Mathlib/RingTheory/Artinian/Module.lean,MathlibTest/LibraryRewrite.lean |
21 |
25 |
['alreadydone', 'artie2000', 'erdOne', 'github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'leanprover-radar'] |
erdOne assignee:erdOne |
0-23084 6 hours ago |
3-69973 3 days ago |
4-55463 4 days |
| 32443 |
vihdzp author:vihdzp |
feat: `SuccOrder` and `PredOrder` instances for `SignType` |
Used in the CGT repo.
---
A future to-do might be to pull out `SuccOrder` and `PredOrder` into a `Defs` file, so that this can be defined within the `Defs` file as well.
[](https://gitpod.io/from-referrer/)
|
t-data |
49/0 |
Mathlib.lean,Mathlib/Data/Sign/SuccPred.lean |
2 |
1 |
['github-actions'] |
nobody |
0-22599 6 hours ago |
0-35766 9 hours ago |
0-35804 9 hours |
| 32408 |
mirefek author:mirefek |
feat(SetTheory/Ordinal): Improve API for Ordinal.toType |
Zulip thread: https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/API.20for.20Ordinal.2EtoType/with/561739587
* Adds coercion from `Ordinal.toType` to `Ordinal` & `Set.Iio o`
* Renames `Ordinal.enumIsoToType` to `Ordinal.toType.mk` with an implicit parameter, so `(.mk ⟨α, h⟩)` can be used to build a `toType`. This prepares for deprecation of the name `Ordinal.enumIsoToType` (to be discussed).
---
[](https://gitpod.io/from-referrer/)
|
t-set-theory
new-contributor
|
47/30 |
Mathlib/SetTheory/Cardinal/Ordinal.lean,Mathlib/SetTheory/Game/Nim.lean,Mathlib/SetTheory/Game/Ordinal.lean,Mathlib/SetTheory/Nimber/Field.lean,Mathlib/SetTheory/Ordinal/Basic.lean,Mathlib/SetTheory/ZFC/Ordinal.lean |
6 |
14 |
['github-actions', 'mirefek', 'vihdzp'] |
nobody |
0-20454 5 hours ago |
1-36703 1 day ago |
1-36744 1 day |
| 31930 |
SnirBroshi author:SnirBroshi |
feat(Data/List/Basic): `idxOf` lemmas |
---
[](https://gitpod.io/from-referrer/)
|
t-data |
29/0 |
Mathlib/Data/List/Basic.lean |
1 |
9 |
['SnirBroshi', 'Vierkantor', 'github-actions'] |
Vierkantor assignee:Vierkantor |
0-19668 5 hours ago |
0-19668 5 hours ago |
11-47522 11 days |
| 32333 |
euprunin author:euprunin |
chore: golf using `grind` |
---
Trace profiling results (shown if ≥10 ms before or after):
* `Set.disjoint_powerset_insert`: <10 ms before, 97 ms after
* `Set.disjoint_image_inl_range_inr`: <10 ms before, 11 ms after
* `Finset.Ico_filter_lt_of_le_right`: <10 ms before, 14 ms after
* `Finset.Ico_filter_le_of_left_le`: <10 ms before, 25 ms after
* `Finset.Ico_filter_le_left`: <10 ms before, 13 ms after
* `Nat.Iio_eq_range`: <10 ms before, 13 ms after
* `Nat.range_eq_Icc_zero_sub_one`: <10 ms before, 32 ms after
* `Nat.Ico_succ_singleton`: <10 ms before, 70 ms after
* `Nat.Ioc_succ_singleton`: <10 ms before, 84 ms after
This golfing PR is batched under the following guidelines:
* Up to 5 changed files per PR
* Up to 25 changed declarations per PR
* Up to 100 changed lines per PR
---
[](https://gitpod.io/from-referrer/)
|
|
15/42 |
Mathlib/Data/Set/Image.lean,Mathlib/Order/Interval/Finset/Basic.lean,Mathlib/Order/Interval/Finset/Nat.lean |
3 |
1 |
['github-actions', 'vihdzp'] |
grunweg assignee:grunweg |
0-19438 5 hours ago |
3-38010 3 days ago |
3-37987 3 days |
| 32451 |
vihdzp author:vihdzp |
chore(Topology/Order/Basic): golf `instIsCountablyGenerated_atTop` |
---
[](https://gitpod.io/from-referrer/)
|
t-topology |
10/22 |
Mathlib/Topology/Order/Basic.lean |
1 |
1 |
['github-actions'] |
nobody |
0-16870 4 hours ago |
0-16873 4 hours ago |
0-16917 4 hours |
| 32452 |
vihdzp author:vihdzp |
chore: add `variable [OrderTopology α]` |
---
[](https://gitpod.io/from-referrer/)
|
t-topology
easy
|
53/57 |
Mathlib/Topology/Order/Basic.lean |
1 |
1 |
['github-actions'] |
nobody |
0-16834 4 hours ago |
0-16892 4 hours ago |
0-16876 4 hours |
| 31471 |
Scarlett-le author:Scarlett-le |
feat(LinearAlgebra/AffineSpace): add commutativity lemmas for line parallelism |
Adds three lemmas showing that parallelism between lines defined by point pairs is invariant under reversing the order of points. |
new-contributor
t-algebra
awaiting-author
label:t-algebra$ |
4/0 |
Mathlib/LinearAlgebra/AffineSpace/AffineSubspace/Basic.lean |
1 |
4 |
['Scarlett-le', 'github-actions', 'mathlib4-merge-conflict-bot', 'ocfnash'] |
ocfnash assignee:ocfnash |
0-16266 4 hours ago |
10-5765 10 days ago |
3-71136 3 days |
| 32453 |
Hagb author:Hagb |
feat(Tactic/WLOG): add `wlog!` a variant of `wlog` that calls `push_neg` |
This commit adds `wlog!`, a variant of the `wlog h : P` tactic that also
calls `push_neg` at the generated hypothesis `h : ¬ p` in the side goal.
---
[](https://gitpod.io/from-referrer/)
|
t-meta |
125/10 |
Mathlib/Tactic/WLOG.lean,MathlibTest/wlog.lean |
2 |
1 |
['github-actions'] |
nobody |
0-16232 4 hours ago |
0-16242 4 hours ago |
0-16281 4 hours |
| 29687 |
vihdzp author:vihdzp |
feat: standard part in non-Archimedean field |
We define `ArchimedeanClass.standardPart x` as the unique real number with an infinitesimal difference from `x`. This generalizes `Hyperreal.st` for a general (non-)archimedean field.
---
- [x] depends on: #29611
- [x] depends on: #29685
- [x] depends on: #29735
- [x] depends on: #30486
- [x] depends on: #32212
[](https://gitpod.io/from-referrer/)
|
t-algebra label:t-algebra$ |
340/15 |
Mathlib.lean,Mathlib/Algebra/Order/CompleteField.lean,Mathlib/Algebra/Order/Ring/Archimedean.lean,Mathlib/Algebra/Ring/Subring/Order.lean,Mathlib/Data/Real/StandardPart.lean,Mathlib/Order/Quotient.lean |
6 |
23 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'plp127', 'vihdzp', 'wwylele'] |
nobody |
0-16171 4 hours ago |
0-16171 4 hours ago |
2-54604 2 days |
| 31730 |
thorimur author:thorimur |
feat(Meta): declaration manipulation meta API: allow logging on type signature of theorems |
This PR introduces some initial definitions in the space of a declaration manipulation meta API.
In the course of #31142, it became apparent that we could benefit from having tools for handling the syntax and elaboration info of user-written declarations.
This PR makes a small beginning towards that end in the Mathlib.Util.DeclarationManipulation module, and provides API for
- getting the info and syntax ref of a declaration given its `Name`
- getting the ref of a theorem's type signature from within some command source syntax given the declaration's ref given above
- running a monadic action with the ambient ref set to that of the type signature of a theorem, with sensible fallbacks
This is used to improve logging locations for the unused-instances-in-types linters, and may be useful for other linters that want to inpsect a theorem's type at the expression level (instead of the syntax level).
(It also introduces the small helper definitions `Syntax.findSome?` and `Syntax.rangeEq`, which behave as expected.)
For context: in the future, it would be nice to
- provide support for all sorts of declarations, not just theorems--but this requires a lot more syntax matching
- provide "exploded views" of declaration syntax like `mkDefView`, but finer grained, and geared for use during linting rather than elaboration
- make it easy to compose complex suggestions to transform different parts of a declaration at once
---
- [x] depends on: #31725
[](https://gitpod.io/from-referrer/)
|
t-meta |
131/0 |
Mathlib.lean,Mathlib/Lean/Syntax.lean,Mathlib/Util/DeclarationManipulation.lean |
3 |
4 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
0-15849 4 hours ago |
0-15870 4 hours ago |
6-61192 6 days |
| 32440 |
thorimur author:thorimur |
bench: erase proofs in types before running `unusedDecidableLinter` |
Checks how much of a performance impact erasing proofs in types has (as opposed to e.g. avoiding them during a traversal, or checking for the presence of our constant, etc.)
---
[](https://gitpod.io/from-referrer/)
|
t-linter |
52/16 |
Mathlib/Tactic/Linter/UnusedInstancesInType.lean,MathlibTest/UnusedInstancesInType.lean |
2 |
3 |
['github-actions', 'leanprover-radar', 'thorimur'] |
nobody |
0-15730 4 hours ago |
0-39543 10 hours ago |
0-0 0 seconds |
| 32450 |
morrison-daniel author:morrison-daniel |
feat(LinearAlgebra/Multilinear): constructing `MultilinearMap` over `DirectSum` |
Adds `fromDirectSumEquiv` as an analog for `fromDFinsuppEquiv` specifically for `DirectSum`. This map combines a collection of `MultilinearMap`s into a single `MultilinearMap` on the `DirectSum`.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-algebra
label:t-algebra$ |
74/0 |
Mathlib.lean,Mathlib/LinearAlgebra/Multilinear/DirectSum.lean |
2 |
n/a |
['github-actions'] |
nobody |
0-14535 4 hours ago |
unknown |
unknown |
| 32374 |
adamtopaz author:adamtopaz |
feat(Tactic/WildcardUniverse): Foo.{*, _, v*, max u v} |
This PR creates an elaborator for syntax of the form `Foo.{*, _, v*, max u v}`. A `*` indicates that a new universe parameter should be created, `_` and `max u v` elaborate using the existing level elaboration (so `_` elaborates to a level mvar). The syntax `v*` creates a level parameter of the form `v_n` for some value of `n`.
The newly created level parameters are ordered in a particular way to match the order in which they appear in the syntax. For example, in `Foo.{*, _, v*, max u v}`, the level parameter associated with `*` will come before the other universes, including the parameter created by `v*`, and the parameters `u` and `v`. Similarly the parameter associated with `v*` will come *after* the one for `*`, and before both `u` and `v`.
Note: Unlike `Category* C`, where we understand exactly how the universes involved in `C` (both in the term and its type) relate to the level parameter of the morphisms, we can't expect such precise control in general. For example, when `C.{u} : Type 0`, `Category* C` places the morphism level `v_1` before `u`, but `Category.{*} C` places it after `u`. In other words, `Foo.{...}` only reorders the level parameters based on the parameters that appear in the (elaborated) `...`, without any regard to the universes that appear in the *arguments* to `Foo.{...}`.
Co-authored-by: Claude
---
[](https://gitpod.io/from-referrer/)
|
t-meta |
656/0 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/WildcardUniverse.lean,MathlibTest/WildcardUniverse.lean |
4 |
22 |
['JovanGerb', 'adamtopaz', 'github-actions'] |
nobody |
0-14058 3 hours ago |
0-32350 8 hours ago |
1-36952 1 day |
| 32455 |
vihdzp author:vihdzp |
feat: order topologies of successor orders |
---
Co-authored by @j-loreaux
[](https://gitpod.io/from-referrer/)
|
t-order
t-topology
|
124/43 |
Mathlib.lean,Mathlib/Order/Cover.lean,Mathlib/SetTheory/Ordinal/Topology.lean,Mathlib/Topology/Order/SuccPred.lean |
4 |
1 |
['github-actions'] |
nobody |
0-13275 3 hours ago |
0-13333 3 hours ago |
0-13325 3 hours |
| 32456 |
morrison-daniel author:morrison-daniel |
feat(LinearAlgebra/Multilinear): interactions of `PiTensorProduct` and `MultilinearMap` |
WIP
---
[](https://gitpod.io/from-referrer/)
|
large-import
new-contributor
t-algebra
WIP
label:t-algebra$ |
211/0 |
Mathlib.lean,Mathlib/LinearAlgebra/DFinsupp/PiTensorProduct.lean,Mathlib/LinearAlgebra/DirectSum/Finsupp.lean,Mathlib/LinearAlgebra/DirectSum/PiTensorProduct.lean |
4 |
n/a |
['github-actions'] |
nobody |
0-12717 3 hours ago |
unknown |
unknown |
| 32030 |
newell author:newell |
feat(Analysis/AperiodicOrder/Delone): Delone Sets |
---
Adds initial definitions and lemmas for Delone Sets.
[](https://gitpod.io/from-referrer/)
|
t-analysis |
199/0 |
Mathlib.lean,Mathlib/Analysis/AperiodicOrder/Delone/Basic.lean |
2 |
30 |
['YaelDillies', 'github-actions', 'j-loreaux', 'newell', 'sgouezel'] |
j-loreaux assignee:j-loreaux |
0-9847 2 hours ago |
1-21002 1 day ago |
6-27854 6 days |
| 31416 |
SnirBroshi author:SnirBroshi |
feat(Combinatorics/SimpleGraph/Walk): lemmas about the first and last darts/edges |
---
[](https://gitpod.io/from-referrer/)
|
t-combinatorics |
67/7 |
Mathlib/Combinatorics/SimpleGraph/Acyclic.lean,Mathlib/Combinatorics/SimpleGraph/Paths.lean,Mathlib/Combinatorics/SimpleGraph/Walks/Basic.lean,Mathlib/Combinatorics/SimpleGraph/Walks/Traversal.lean |
4 |
7 |
['SnirBroshi', 'YaelDillies', 'github-actions', 'mathlib4-merge-conflict-bot'] |
YaelDillies assignee:YaelDillies |
0-9569 2 hours ago |
0-21068 5 hours ago |
20-51720 20 days |
| 32412 |
Brian-Nugent author:Brian-Nugent |
feat: add Artinian schemes |
Added the definition of Artinian Schemes and proved basic facts about them.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-algebraic-geometry
awaiting-author
|
152/0 |
Mathlib.lean,Mathlib/AlgebraicGeometry/Artinian.lean |
2 |
31 |
['Brian-Nugent', 'erdOne', 'github-actions'] |
erdOne assignee:erdOne |
0-7257 2 hours ago |
1-15767 1 day ago |
0-5367 1 hour |
| 30622 |
kim-em author:kim-em |
feat: replace some tauto with grind |
This PR replaces an initial segment of `tauto` calls with `grind`. Note that not all `tauto` calls are replaceable, as (amongst other smaller issues) `tauto` is willing to unfold things `grind` won't. |
awaiting-author |
33/33 |
Archive/Examples/Kuratowski.lean,Archive/Imo/Imo2001Q3.lean,Counterexamples/Phillips.lean,Mathlib/Algebra/BigOperators/Intervals.lean,Mathlib/Algebra/CubicDiscriminant.lean,Mathlib/Algebra/Group/Int/Units.lean,Mathlib/Algebra/Group/Subgroup/Basic.lean,Mathlib/Algebra/Group/Subgroup/Lattice.lean,Mathlib/Algebra/GroupWithZero/Indicator.lean,Mathlib/Algebra/Homology/Double.lean,Mathlib/Algebra/Homology/HomotopyCategory/MappingCone.lean,Mathlib/Algebra/Homology/HomotopyCofiber.lean,Mathlib/Algebra/Homology/ShortComplex/Ab.lean,Mathlib/Algebra/Homology/ShortComplex/ModuleCat.lean,Mathlib/Algebra/Lie/Derivation/AdjointAction.lean,Mathlib/Algebra/Lie/Nilpotent.lean,Mathlib/Algebra/Lie/Weights/Killing.lean,Mathlib/Algebra/Module/Torsion/Basic.lean,Mathlib/Algebra/Order/GroupWithZero/Canonical.lean,Mathlib/Algebra/Polynomial/Homogenize.lean,Mathlib/Algebra/Ring/NegOnePow.lean,Mathlib/AlgebraicGeometry/EllipticCurve/IsomOfJ.lean,Mathlib/AlgebraicGeometry/ValuativeCriterion.lean,Mathlib/AlgebraicTopology/DoldKan/NReflectsIso.lean,Mathlib/AlgebraicTopology/SimplicialSet/Simplices.lean,Mathlib/Analysis/Analytic/IsolatedZeros.lean |
26 |
7 |
['github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'mathlib4-merge-conflict-bot', 'ocfnash', 'urkud'] |
mattrobball assignee:mattrobball |
0-4761 1 hour ago |
0-4761 1 hour ago |
11-29633 11 days |
| 29776 |
yuanyi-350 author:yuanyi-350 |
chore: refactor `ContinuousLinearMap.isOpenMap` by separating it into sublemmas |
The open mapping theorem in mathlib proves A ⇒ C by first proving A ⇒ B and then B ⇒ C in one theorem. In my PR, I separated it into two theorems: A ⇒ B and B ⇒ C. And now B ⇒ C is more general, with weaker assumptions than A ⇒ C.
The [open mapping theorem](https://leanprover-community.github.io/mathlib4_docs/Mathlib/Analysis/Normed/Operator/Banach.html#ContinuousLinearMap.isOpenMap) in mathlib need `f` to be surjective.
However, this can be weakened to the condition `h : ∃ (n : ℕ) (x : _), x ∈ interior (closure (f '' ball 0 n))` . I need this stronger formulation to prove the closed range theorem c.f. *Rudin Functional Analysis Thm 4.13*
[zulip](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/refactor.20.60ContinuousLinearMap.2EisOpenMap.60)
---
[](https://gitpod.io/from-referrer/)
|
t-analysis
WIP
|
55/35 |
Mathlib/Analysis/Normed/Operator/Banach.lean |
1 |
15 |
['faenuccio', 'github-actions', 'kckennylau', 'leanprover-bot', 'themathqueen', 'yuanyi-350'] |
faenuccio assignee:faenuccio |
0-4213 1 hour ago |
0-23391 6 hours ago |
2-46827 2 days |
| 32458 |
vihdzp author:vihdzp |
feat: order isomorphisms preserve successor/predecessor limits |
---
Co-authored by: Aaron Liu @plp127
[](https://gitpod.io/from-referrer/)
|
t-order |
31/1 |
Mathlib/Order/SuccPred/Limit.lean |
1 |
1 |
['github-actions'] |
nobody |
0-3995 1 hour ago |
0-4033 1 hour ago |
0-4038 1 hour |
| 32460 |
loefflerd author:loefflerd |
feat(ModularForms): norm and trace maps |
Define norm and trace maps from modular forms for a finite-index inclusion of levels, and use these to show that modular forms of negative weight are 0 for any arithmetic subgroup.
---
[](https://gitpod.io/from-referrer/)
|
t-number-theory |
272/0 |
Mathlib.lean,Mathlib/NumberTheory/ModularForms/NormTrace.lean |
2 |
1 |
['github-actions'] |
nobody |
0-1988 33 minutes ago |
0-1993 32 minutes ago |
0-2035 33 minutes |
| 31802 |
joelriou author:joelriou |
feat(AlgebraicTopology): horns in `Δ[2]` as pushouts |
Horns in `Δ[2]` are pushouts of two copies of `Δ[1]`.
Co-authored-by: Nick Ward
From https://github.com/joelriou/topcat-model-category
---
- [x] depends on: #31797
[](https://gitpod.io/from-referrer/)
|
t-algebraic-topology |
244/0 |
Mathlib.lean,Mathlib/AlgebraicTopology/SimplicialSet/Horn.lean,Mathlib/AlgebraicTopology/SimplicialSet/HornColimits.lean,Mathlib/AlgebraicTopology/SimplicialSet/StdSimplex.lean,Mathlib/AlgebraicTopology/SimplicialSet/Subcomplex.lean,Mathlib/CategoryTheory/Limits/Shapes/Pullback/CommSq.lean |
6 |
3 |
['github-actions', 'joelriou', 'mathlib4-dependent-issues-bot'] |
robin-carlier assignee:robin-carlier |
0-1824 30 minutes ago |
7-78356 7 days ago |
7-78334 7 days |
| 32461 |
joelriou author:joelriou |
feat(Algebra/Homology): more API for the HomComplex from a single cochain complex |
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebra
t-category-theory
label:t-algebra$ |
111/16 |
Mathlib/Algebra/Homology/HomotopyCategory/HomComplex.lean,Mathlib/Algebra/Homology/HomotopyCategory/HomComplexCohomology.lean,Mathlib/Algebra/Homology/HomotopyCategory/HomComplexSingle.lean |
3 |
1 |
['github-actions'] |
nobody |
0-1795 29 minutes ago |
0-1890 31 minutes ago |
0-1937 32 minutes |
| 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
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 |
0-1679 27 minutes ago |
153-11903 5 months ago |
0-135 2 minutes |
| 32316 |
Thmoas-Guan author:Thmoas-Guan |
feat(Homology/ModuleCat): Dimension Shifting tools in ModuleCat |
In this PR we present some dimension shifting tools in `ModuleCat`.
---
- [x] depends on: #32312
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-category-theory
awaiting-author
label:t-algebra$ |
124/0 |
Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Ext/DimensionShifting.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/EnoughInjectives.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/EnoughProjectives.lean |
4 |
10 |
['Thmoas-Guan', 'github-actions', 'jcommelin', 'joelriou', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
joelriou assignee:joelriou |
0-1339 22 minutes ago |
0-41378 11 hours ago |
0-25818 7 hours |
| 32252 |
ajirving author:ajirving |
feat(NumberTheory.Chebyshev): prove relationship between psi and theta |
Proves the relationship between the Chebyshev psi and theta functions; psi is a sum of theta evaluated at powers of x. This upstreams a result from the PrimeNumberTheoremAnd pproject.
---
- [x] depends on: #32247
[](https://gitpod.io/from-referrer/)
|
large-import
new-contributor
t-number-theory
|
200/2 |
Mathlib/NumberTheory/Chebyshev.lean |
1 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
0-979 16 minutes ago |
0-50836 14 hours ago |
0-56667 15 hours |
| 32459 |
vihdzp author:vihdzp |
chore(Order/Directed): use `to_dual` |
I've made an effort to dualize specifically lemmas about `IsDirected α (· ≤ ·)`, so as to reduce the number of appearances of ≥ in code.
---
[](https://gitpod.io/from-referrer/)
|
t-order
awaiting-CI
|
23/48 |
Mathlib/Order/Directed.lean,Mathlib/Topology/DiscreteQuotient.lean |
2 |
1 |
['github-actions'] |
nobody |
0-946 15 minutes ago |
0-946 15 minutes ago |
0-0 0 seconds |
| 32447 |
vihdzp author:vihdzp |
chore(Order/SuccPred/Basic): use `to_dual` |
Not everything has been dualized yet. Dualizing theorems about `Monotone`, `Ixx`, `Order(Bot/Top)` still depends on other PRs.
---
[](https://gitpod.io/from-referrer/)
|
t-order |
98/171 |
Mathlib/Order/Interval/Set/SuccPred.lean,Mathlib/Order/Iterate.lean,Mathlib/Order/SuccPred/Basic.lean,Mathlib/Tactic/Translate/ToDual.lean |
4 |
7 |
['JovanGerb', 'github-actions', 'vihdzp'] |
nobody |
0-887 14 minutes ago |
0-13720 3 hours ago |
0-13706 3 hours |
| 32457 |
vihdzp author:vihdzp |
chore: mark `Set.not_finite` as `simp` |
---
[](https://gitpod.io/from-referrer/)
|
t-data |
2/2 |
Mathlib/Data/Finite/Defs.lean |
1 |
1 |
['github-actions'] |
nobody |
0-821 13 minutes ago |
0-821 13 minutes ago |
0-820 13 minutes |
| 32462 |
vihdzp author:vihdzp |
refactor: make `abbrev`s for `IsDirected α (· ≤ ·)` and `IsDirected α (· ≥ ·)` |
This standardizes how we write these typeclasses, and lets us use the `to_dual` tactic in the future.
---
[](https://gitpod.io/from-referrer/)
|
t-order
awaiting-CI
|
193/191 |
Mathlib/Algebra/Colimit/DirectLimit.lean,Mathlib/Algebra/Colimit/Finiteness.lean,Mathlib/Algebra/Colimit/Module.lean,Mathlib/Algebra/Colimit/Ring.lean,Mathlib/Algebra/Order/Archimedean/Basic.lean,Mathlib/Algebra/Order/Group/Indicator.lean,Mathlib/Analysis/Convex/Quasiconvex.lean,Mathlib/Analysis/Normed/Ring/Basic.lean,Mathlib/CategoryTheory/CofilteredSystem.lean,Mathlib/CategoryTheory/Filtered/Basic.lean,Mathlib/CategoryTheory/Filtered/Final.lean,Mathlib/CategoryTheory/Presentable/Type.lean,Mathlib/Data/ENNReal/BigOperators.lean,Mathlib/Data/ENNReal/Operations.lean,Mathlib/Data/ENat/BigOperators.lean,Mathlib/Data/ENat/Lattice.lean,Mathlib/Data/Finset/Basic.lean,Mathlib/Data/Finset/Order.lean,Mathlib/Data/Fintype/Order.lean,Mathlib/Data/Set/Finite/Lattice.lean,Mathlib/Data/Set/Lattice.lean,Mathlib/MeasureTheory/Function/SimpleFunc.lean,Mathlib/MeasureTheory/Integral/IntegrableOn.lean,Mathlib/MeasureTheory/MeasurableSpace/MeasurablyGenerated.lean,Mathlib/MeasureTheory/Measure/MeasureSpace.lean,Mathlib/ModelTheory/DirectLimit.lean,Mathlib/ModelTheory/Fraisse.lean,Mathlib/ModelTheory/PartialEquiv.lean,Mathlib/Order/Bounds/Basic.lean,Mathlib/Order/CompleteBooleanAlgebra.lean,Mathlib/Order/Directed.lean,Mathlib/Order/DirectedInverseSystem.lean,Mathlib/Order/Filter/AtTopBot/Archimedean.lean,Mathlib/Order/Filter/AtTopBot/Basic.lean,Mathlib/Order/Filter/AtTopBot/CountablyGenerated.lean,Mathlib/Order/Filter/AtTopBot/Finset.lean,Mathlib/Order/Filter/AtTopBot/Prod.lean,Mathlib/Order/Filter/Bases/Basic.lean,Mathlib/Order/Filter/CountablyGenerated.lean,Mathlib/Order/Filter/IsBounded.lean,Mathlib/Order/Ideal.lean,Mathlib/Order/SuccPred/Archimedean.lean,Mathlib/Topology/Algebra/InfiniteSum/SummationFilter.lean,Mathlib/Topology/Category/TopCat/Limits/Konig.lean,Mathlib/Topology/Order/LiminfLimsup.lean,Mathlib/Topology/UniformSpace/UniformConvergenceTopology.lean |
46 |
1 |
['github-actions'] |
nobody |
0-298 4 minutes ago |
0-851 13 minutes ago |
0-13 13 seconds |
| 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
WIP
|
2225/6 |
Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Ext/DimensionShifting.lean,Mathlib/Algebra/Category/ModuleCat/Ext/Finite.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/EnoughInjectives.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/EnoughProjectives.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/RingTheory/CohenMacaulay/Basic.lean,Mathlib/RingTheory/CohenMacaulay/Polynomial.lean,Mathlib/RingTheory/Regular/Category.lean,Mathlib/RingTheory/Regular/Depth.lean,Mathlib/RingTheory/Regular/Ischebeck.lean |
11 |
n/a |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
0-285 4 minutes ago |
unknown |
unknown |
| 32449 |
vihdzp author:vihdzp |
refactor: `Ordinal.toType` → `Ordinal.ToType` |
See [Zulip](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/toType.20capitalization/with/562007379).
---
[](https://gitpod.io/from-referrer/)
|
t-set-theory
awaiting-CI
|
145/142 |
Mathlib/CategoryTheory/Abelian/GrothendieckCategory/EnoughInjectives.lean,Mathlib/CategoryTheory/Presentable/CardinalFilteredPresentation.lean,Mathlib/CategoryTheory/Presentable/IsCardinalFiltered.lean,Mathlib/CategoryTheory/Presentable/OrthogonalReflection.lean,Mathlib/CategoryTheory/SmallObject/Basic.lean,Mathlib/CategoryTheory/SmallObject/IsCardinalForSmallObjectArgument.lean,Mathlib/CategoryTheory/SmallRepresentatives.lean,Mathlib/FieldTheory/CardinalEmb.lean,Mathlib/SetTheory/Cardinal/Cofinality.lean,Mathlib/SetTheory/Cardinal/Regular.lean,Mathlib/SetTheory/Game/Nim.lean,Mathlib/SetTheory/Game/Ordinal.lean,Mathlib/SetTheory/Nimber/Field.lean,Mathlib/SetTheory/Ordinal/Arithmetic.lean,Mathlib/SetTheory/Ordinal/Basic.lean,Mathlib/SetTheory/Ordinal/Family.lean,Mathlib/SetTheory/ZFC/Ordinal.lean |
17 |
1 |
['github-actions'] |
nobody |
0-259 4 minutes ago |
0-4448 1 hour ago |
0-10 10 seconds |
| 31558 |
AntoineChambert-Loir author:AntoineChambert-Loir |
feat(Topology/Sublevel): sublevels in relation with semicontinuity and compactness |
Two lemmas about sublevels and semicontinuity related to compactness
* `Set.isCompact_inter_preimage_Iic`, the sublevels of a lower semicontinuous function on a compact set are compact.
* `Set.biInter_sep_map_le_eq_empty_iff_exists_finset`, an intersection of sublevel sets of a lower semicontinuous function on a compact set is empty if and only if a finite sub-intersection is already empty.
Co-authored with @ADedecker
---
[](https://gitpod.io/from-referrer/)
|
t-topology |
61/0 |
Mathlib/Topology/Compactness/Compact.lean,Mathlib/Topology/Semicontinuous.lean |
2 |
32 |
['AntoineChambert-Loir', 'github-actions', 'j-loreaux', 'mathlib4-merge-conflict-bot'] |
j-loreaux assignee:j-loreaux |
0-250 4 minutes ago |
2-58350 2 days ago |
16-8272 16 days |
| 32407 |
harahu author:harahu |
doc: fix typos found by codespell |
Typos found by running codespell. Fixed with help from Codex.
---
[](https://gitpod.io/from-referrer/)
|
|
58/58 |
Archive/Examples/Kuratowski.lean,Mathlib/Algebra/Group/Int/Defs.lean,Mathlib/Algebra/MonoidAlgebra/Basic.lean,Mathlib/Algebra/SkewPolynomial/Basic.lean,Mathlib/Analysis/Distribution/TestFunction.lean,Mathlib/CategoryTheory/Bicategory/Functor/StrictPseudofunctor.lean,Mathlib/CategoryTheory/ConcreteCategory/BundledHom.lean,Mathlib/CategoryTheory/ConcreteCategory/UnbundledHom.lean,Mathlib/CategoryTheory/Sites/Descent/IsPrestack.lean,Mathlib/CategoryTheory/Sites/Point/Basic.lean,Mathlib/Combinatorics/SimpleGraph/Connectivity/Connected.lean,Mathlib/Data/Fin/Tuple/Basic.lean,Mathlib/Data/List/Chain.lean,Mathlib/Geometry/Manifold/Immersion.lean,Mathlib/Geometry/Manifold/SmoothApprox.lean,Mathlib/GroupTheory/FreeGroup/Orbit.lean,Mathlib/LinearAlgebra/Contraction.lean,Mathlib/LinearAlgebra/Matrix/PosDef.lean,Mathlib/LinearAlgebra/SpecialLinearGroup.lean,Mathlib/LinearAlgebra/SymmetricAlgebra/Basic.lean,Mathlib/MeasureTheory/Integral/CurveIntegral/Basic.lean,Mathlib/NumberTheory/ModularForms/EisensteinSeries/QExpansion.lean,Mathlib/Order/Lattice/Congruence.lean,Mathlib/Probability/Independence/BoundedContinuousFunction.lean,Mathlib/Probability/Independence/CharacteristicFunction.lean,Mathlib/Probability/Martingale/Basic.lean,Mathlib/RingTheory/Congruence/Hom.lean,Mathlib/RingTheory/Extension/Presentation/Basic.lean,Mathlib/Tactic/Order/ToInt.lean,Mathlib/Tactic/Simproc/ExistsAndEq.lean,Mathlib/Tactic/Translate/Core.lean,Mathlib/Tactic/Translate/ToDual.lean,Mathlib/Topology/Algebra/IsUniformGroup/Defs.lean,Mathlib/Topology/Algebra/Module/PointwiseConvergence.lean,Mathlib/Topology/CWComplex/Classical/Subcomplex.lean,Mathlib/Topology/EMetricSpace/PairReduction.lean,Mathlib/Topology/Homotopy/LocallyContractible.lean,MathlibTest/EmptyLine.lean,MathlibTest/FieldSimp.lean,MathlibTest/ImportHeavyFlexibleLinter.lean,MathlibTest/ToDual.lean,MathlibTest/grind/lint.lean |
42 |
1 |
['github-actions'] |
nobody |
0-108 1 minute ago |
1-38511 1 day ago |
1-42742 1 day |
| 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 |
492-69 1 year ago |
505-77464 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 |
492-68 1 year ago |
525-26765 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 |
492-68 1 year ago |
529-84759 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 |
492-68 1 year ago |
504-74079 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 |
492-67 1 year ago |
533-81249 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 |
492-67 1 year ago |
503-64198 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 |
492-67 1 year ago |
533-81376 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 |
492-66 1 year ago |
562-208 1 year ago |
0-0 0 seconds |
| 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 |
492-66 1 year ago |
513-67166 1 year ago |
0-0 0 seconds |
| 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 |
492-66 1 year ago |
580-62257 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 |
492-66 1 year ago |
559-52458 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 |
492-66 1 year ago |
505-9663 1 year ago |
1-73101 1 day |
| 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 |
492-66 1 year ago |
505-9657 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 |
492-66 1 year ago |
584-2064 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 |
492-66 1 year ago |
580-3642 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 |
492-66 1 year ago |
540-81530 1 year ago |
5-72414 5 days |
| 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 |
492-66 1 year ago |
549-45611 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 |
492-66 1 year ago |
562-209 1 year ago |
0-0 0 seconds |
| 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 |
492-65 1 year ago |
503-64332 1 year ago |
1-21749 1 day |
| 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 |
492-65 1 year ago |
614-38195 1 year ago |
1-12270 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 |
492-64 1 year ago |
503-64921 1 year ago |
0-832 13 minutes |
| 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 |
492-64 1 year ago |
553-23723 1 year ago |
0-0 0 seconds |
| 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 |
492-64 1 year ago |
513-67166 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 |
492-64 1 year ago |
647-24597 1 year ago |
0-0 0 seconds |
| 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 |
492-64 1 year ago |
599-14126 1 year ago |
1-29105 1 day |
| 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 |
492-64 1 year ago |
513-67166 1 year ago |
64-12826 64 days |
| 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 |
492-63 1 year ago |
694-10361 1 year ago |
38-46649 38 days |
| 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 |
492-63 1 year ago |
640-58778 1 year ago |
5-6524 5 days |
| 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 |
492-63 1 year ago |
742-73319 2 years 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 |
492-63 1 year ago |
541-65117 1 year ago |
29-65537 29 days |
| 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 |
492-63 1 year ago |
496-81532 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 |
492-63 1 year ago |
675-20460 1 year ago |
19-26304 19 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 |
492-63 1 year ago |
743-5241 2 years 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 |
492-63 1 year ago |
513-67166 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 |
492-63 1 year ago |
525-74365 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 |
492-63 1 year ago |
593-36192 1 year ago |
0-0 0 seconds |
| 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 |
492-63 1 year ago |
673-8191 1 year ago |
7-6153 7 days |
| 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 |
492-63 1 year ago |
679-78707 1 year ago |
0-0 0 seconds |
| 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 |
492-63 1 year ago |
669-66365 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 |
492-63 1 year ago |
622-53152 1 year ago |
22-72922 22 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 |
492-63 1 year ago |
550-43488 1 year ago |
0-0 0 seconds |
| 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 |
492-63 1 year ago |
680-3912 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 |
492-63 1 year ago |
584-76669 1 year ago |
0-0 0 seconds |
| 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 |
492-63 1 year ago |
580-61247 1 year ago |
0-0 0 seconds |
| 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 |
492-63 1 year ago |
655-76180 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 |
492-62 1 year ago |
503-65179 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 |
492-62 1 year ago |
512-39921 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 |
492-62 1 year ago |
621-49728 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 |
492-62 1 year ago |
694-67898 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 |
492-62 1 year ago |
513-67166 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 |
492-62 1 year ago |
513-67166 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 |
492-62 1 year ago |
767-26503 2 years ago |
0-72515 20 hours |
| 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 |
492-62 1 year ago |
513-67166 1 year ago |
0-0 0 seconds |
| 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 |
492-62 1 year ago |
513-67166 1 year ago |
1-47913 1 day |
| 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 |
492-62 1 year ago |
608-74894 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 |
492-62 1 year ago |
822-60485 2 years 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 |
492-62 1 year ago |
653-35474 1 year 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 |
492-62 1 year ago |
766-5902 2 years ago |
0-62955 17 hours |
| 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 |
492-62 1 year ago |
685-65367 1 year ago |
0-0 0 seconds |
| 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 |
492-62 1 year ago |
808-54322 2 years ago |
0-0 0 seconds |
| 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 |
492-62 1 year ago |
549-11054 1 year ago |
0-0 0 seconds |
| 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 |
492-62 1 year ago |
503-65051 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 |
492-62 1 year ago |
513-67166 1 year ago |
35-56459 35 days |
| 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 |
492-61 1 year ago |
507-12890 1 year ago |
0-0 0 seconds |
| 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 |
492-61 1 year ago |
530-82272 1 year ago |
43-56043 43 days |
| 6403 |
astrainfinita author:astrainfinita |
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 |
['Vierkantor', 'astrainfinita', 'digama0', 'eric-wieser', 'j-loreaux', 'leanprover-bot'] |
nobody |
492-61 1 year ago |
550-43531 1 year ago |
13-18399 13 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 |
492-61 1 year ago |
513-67166 1 year ago |
0-0 0 seconds |
| 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 |
492-61 1 year ago |
513-67166 1 year ago |
5-55287 5 days |
| 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 |
492-61 1 year ago |
756-76058 2 years ago |
9-67365 9 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 |
492-61 1 year ago |
532-83889 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 |
492-61 1 year ago |
842-54102 2 years 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 |
492-61 1 year ago |
661-73450 1 year ago |
0-0 0 seconds |
| 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 |
492-61 1 year ago |
766-6669 2 years 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 |
492-61 1 year ago |
843-3198 2 years ago |
0-4269 1 hour |
| 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 |
492-61 1 year ago |
513-67166 1 year ago |
83-76369 83 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 |
492-61 1 year ago |
838-47986 2 years ago |
0-19160 5 hours |
| 6330 |
astrainfinita author:astrainfinita |
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 |
['astrainfinita', 'digama0', 'leanprover-bot'] |
nobody |
492-61 1 year ago |
550-43551 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 |
492-61 1 year ago |
513-67166 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 |
492-61 1 year ago |
513-67166 1 year 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 |
492-61 1 year ago |
523-60056 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 |
492-61 1 year ago |
814-19436 2 years ago |
0-0 0 seconds |
| 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 |
492-61 1 year ago |
912-11377 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 |
492-61 1 year ago |
847-38325 2 years 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 |
492-60 1 year ago |
744-11246 2 years 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 |
487-62770 1 year ago |
487-62770 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 |
484-74439 1 year ago |
484-74439 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 |
479-67533 1 year ago |
485-18155 1 year ago |
0-0 0 seconds |
| 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 |
479-43615 1 year ago |
479-43615 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 |
477-80006 1 year ago |
477-80006 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 |
477-79539 1 year ago |
477-79539 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 |
477-77938 1 year ago |
477-77938 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 |
477-64702 1 year ago |
477-64702 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 |
476-76723 1 year ago |
476-76723 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 |
476-76520 1 year ago |
476-76520 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 |
476-76383 1 year ago |
476-76383 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 |
476-76368 1 year ago |
476-76368 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 |
476-76330 1 year ago |
476-76330 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 |
476-76306 1 year ago |
476-76306 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 |
476-76296 1 year ago |
476-76296 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 |
476-76215 1 year ago |
476-76215 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 |
476-76180 1 year ago |
476-76180 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 |
476-76148 1 year ago |
476-76148 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 |
476-76002 1 year ago |
476-76002 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 |
476-75825 1 year ago |
476-75825 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 |
476-75767 1 year ago |
476-75767 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 |
476-75712 1 year ago |
476-75712 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 |
476-75706 1 year ago |
476-75706 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 |
476-75574 1 year ago |
476-75574 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 |
475-21582 1 year ago |
475-21582 1 year ago |
0-0 0 seconds |
| 15586 |
astrainfinita author:astrainfinita |
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 |
['astrainfinita', 'github-actions', 'leanprover-bot'] |
nobody |
475-21582 1 year ago |
475-21582 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 |
473-42851 1 year ago |
513-67166 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 |
473-42710 1 year ago |
513-67166 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 |
473-42609 1 year ago |
513-67166 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 |
473-42401 1 year ago |
473-42401 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 |
473-41712 1 year ago |
473-41712 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 |
473-20275 1 year ago |
473-20275 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 |
472-83799 1 year ago |
473-1313 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 |
472-63763 1 year ago |
477-80005 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 |
472-52816 1 year ago |
473-41963 1 year ago |
7-18420 7 days |
| 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 |
470-66037 1 year ago |
477-80007 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 |
470-66017 1 year ago |
476-76612 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 |
470-65855 1 year ago |
549-55445 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 |
464-79459 1 year ago |
464-79459 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 |
463-47735 1 year ago |
463-47735 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 |
461-70949 1 year ago |
461-70950 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 |
461-69937 1 year ago |
461-69937 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 |
457-63451 1 year ago |
457-63451 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 |
457-63451 1 year ago |
457-63451 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 |
452-58195 1 year ago |
452-58198 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 |
452-18332 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 |
450-83088 1 year ago |
450-83088 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 |
450-12224 1 year ago |
450-12224 1 year ago |
32-30254 32 days |
| 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 |
446-41157 1 year ago |
446-41157 1 year 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 |
446-21457 1 year ago |
446-21457 1 year ago |
0-0 0 seconds |
| 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 |
443-78411 1 year ago |
443-78411 1 year 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 |
441-67020 1 year ago |
441-67020 1 year ago |
0-14835 4 hours |
| 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 |
441-4274 1 year ago |
441-4274 1 year 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 |
440-52319 1 year ago |
440-52319 1 year 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 |
437-2906 1 year ago |
437-2907 1 year ago |
21-9462 21 days |
| 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 |
432-47999 1 year ago |
432-47999 1 year 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 |
431-19659 1 year ago |
431-19659 1 year 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 |
431-14702 1 year ago |
431-14702 1 year 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 |
424-77655 1 year ago |
427-14731 1 year 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 |
423-13198 1 year ago |
423-13198 1 year 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 |
421-59844 1 year ago |
421-59844 1 year 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 |
421-43507 1 year ago |
513-67166 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 |
419-5785 1 year ago |
503-63929 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 |
416-66984 1 year ago |
416-66984 1 year 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 |
416-66608 1 year ago |
416-66608 1 year 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 |
413-2648 1 year ago |
413-2648 1 year 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 |
408-64833 1 year ago |
408-64833 1 year 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 |
407-36415 1 year ago |
407-36415 1 year 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 |
405-85307 1 year ago |
405-85307 1 year 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 |
400-39602 1 year ago |
427-8393 1 year 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 |
396-26259 1 year ago |
396-26259 1 year 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 |
396-26013 1 year ago |
396-26013 1 year 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 |
396-4570 1 year ago |
396-4570 1 year 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 |
395-38767 1 year ago |
395-38767 1 year 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 |
395-29521 1 year ago |
395-29535 1 year 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 |
394-64980 1 year ago |
513-67166 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 |
394-10168 1 year ago |
394-10168 1 year 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 |
394-9071 1 year ago |
394-9071 1 year 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 |
392-83839 1 year ago |
392-83839 1 year 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 |
391-52689 1 year ago |
391-52689 1 year 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 |
388-18112 1 year 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 |
387-5121 1 year 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 |
386-66654 1 year ago |
386-66654 1 year 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 |
385-75914 1 year ago |
385-75914 1 year 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 |
384-85668 1 year ago |
384-85668 1 year 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 |
384-84906 1 year ago |
384-84906 1 year 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 |
384-41167 1 year ago |
384-41167 1 year 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 |
383-84602 1 year ago |
383-84602 1 year 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 |
381-66360 1 year ago |
381-66360 1 year 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 |
381-61888 1 year ago |
674-84361 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 |
381-43531 1 year ago |
381-43531 1 year 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 |
380-48542 1 year ago |
380-48542 1 year 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 |
379-71884 1 year ago |
379-71884 1 year 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 |
378-9136 1 year ago |
378-9136 1 year ago |
0-0 0 seconds |
| 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 |
374-68078 1 year ago |
374-68078 1 year 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 |
373-73323 1 year ago |
373-73323 1 year 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 |
371-49400 1 year ago |
371-49400 1 year ago |
4-60621 4 days |
| 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 |
367-76747 1 year ago |
476-75937 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 |
364-80405 11 months ago |
364-80405 11 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 |
360-15069 11 months ago |
360-15069 11 months ago |
31-75259 31 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 |
357-27538 11 months ago |
363-62961 11 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 |
355-74864 11 months ago |
355-74864 11 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 |
353-65482 11 months ago |
353-65485 11 months ago |
0-989 16 minutes |
| 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 |
349-84684 11 months ago |
349-84684 11 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 |
349-84683 11 months ago |
349-84683 11 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 |
344-65876 11 months ago |
344-65877 11 months ago |
0-0 0 seconds |
| 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 |
336-39050 11 months ago |
336-39050 11 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 |
334-13703 11 months ago |
334-13703 11 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 |
334-13702 11 months ago |
334-13702 11 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 |
332-31243 10 months ago |
332-31243 10 months ago |
135-29017 135 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 |
323-49550 10 months ago |
323-49550 10 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 |
323-49305 10 months ago |
323-49305 10 months ago |
76-67978 76 days |
| 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 |
322-68636 10 months ago |
322-68636 10 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 |
322-34555 10 months ago |
322-34555 10 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 |
320-41809 10 months ago |
320-41809 10 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 |
320-26405 10 months ago |
320-26405 10 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 |
317-56214 10 months ago |
317-56215 10 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 |
315-85425 10 months ago |
315-85425 10 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 |
310-73562 10 months ago |
310-73562 10 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 |
309-47995 10 months ago |
309-47995 10 months ago |
9-73631 9 days |
| 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 |
308-64155 10 months ago |
743-37442 2 years 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 |
308-41660 10 months ago |
308-41660 10 months ago |
101-64856 101 days |
| 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 |
303-6339 10 months ago |
303-6339 10 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 |
301-67556 9 months ago |
301-67556 9 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 |
300-48757 9 months ago |
300-48757 9 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 |
299-47878 9 months ago |
299-47878 9 months ago |
0-7781 2 hours |
| 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 |
297-42289 9 months ago |
297-42289 9 months ago |
17-44773 17 days |
| 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 |
295-58799 9 months ago |
295-58799 9 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 |
293-85423 9 months ago |
293-85423 9 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 |
293-65218 9 months ago |
293-65218 9 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 |
293-64971 9 months ago |
293-64971 9 months ago |
37-29014 37 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 |
291-11927 9 months ago |
367-5109 1 year 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 |
290-49544 9 months ago |
290-49544 9 months ago |
0-0 0 seconds |
| 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 |
288-21399 9 months ago |
288-21399 9 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 |
287-75106 9 months ago |
287-75106 9 months ago |
195-56460 195 days |
| 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 |
281-39007 9 months ago |
281-39008 9 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 |
280-38638 9 months ago |
280-38638 9 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 |
279-73569 9 months ago |
279-73569 9 months ago |
125-12755 125 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 |
278-51600 9 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 |
276-74690 9 months ago |
276-74690 9 months ago |
0-0 0 seconds |
| 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 |
272-61596 8 months ago |
272-61596 8 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 |
270-31010 8 months ago |
270-31010 8 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 |
269-23886 8 months ago |
269-23886 8 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 |
268-55079 8 months ago |
268-55079 8 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 |
267-30742 8 months ago |
448-83092 1 year ago |
119-35643 119 days |
| 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 |
266-55409 8 months ago |
266-55409 8 months ago |
29-48368 29 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 |
262-27472 8 months ago |
262-27472 8 months ago |
7-47472 7 days |
| 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 |
260-49505 8 months ago |
260-49505 8 months ago |
3-28829 3 days |
| 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 |
259-19138 8 months ago |
259-19138 8 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 |
257-68541 8 months ago |
257-68542 8 months ago |
22-71271 22 days |
| 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 |
253-26073 8 months ago |
253-26073 8 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 |
252-48825 8 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 |
252-5266 8 months ago |
252-5266 8 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 |
251-60622 8 months ago |
251-60622 8 months ago |
0-0 0 seconds |
| 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 |
246-8277 8 months ago |
246-8277 8 months ago |
0-1769 29 minutes |
| 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 |
244-63999 8 months ago |
244-63999 8 months ago |
0-214 3 minutes |
| 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 |
242-85797 7 months ago |
242-85797 7 months ago |
51-85104 51 days |
| 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 |
241-17769 7 months ago |
241-17772 7 months ago |
0-0 0 seconds |
| 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 |
239-72206 7 months ago |
239-72207 7 months ago |
0-0 0 seconds |
| 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 |
239-12421 7 months ago |
239-12423 7 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 |
238-80517 7 months ago |
238-80519 7 months ago |
4-16654 4 days |
| 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 |
237-65178 7 months ago |
237-65180 7 months ago |
1-44375 1 day |
| 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 |
234-6549 7 months ago |
234-6551 7 months ago |
55-52030 55 days |
| 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 |
233-38202 7 months ago |
503-64792 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 |
233-38081 7 months ago |
513-67166 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 |
233-38056 7 months ago |
503-65051 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 |
233-37882 7 months ago |
513-67166 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 |
233-37842 7 months ago |
481-76172 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 |
233-37618 7 months ago |
437-77165 1 year 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 |
233-5132 7 months ago |
528-74876 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 |
233-4684 7 months ago |
631-35356 1 year ago |
0-0 0 seconds |
| 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 |
231-41911 7 months ago |
231-41911 7 months ago |
25-60481 25 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 |
229-60421 7 months ago |
229-60423 7 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 |
229-55036 7 months ago |
515-68962 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 |
226-84883 7 months ago |
unknown |
unknown |
| 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 |
224-27261 7 months ago |
235-55891 7 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 |
222-58788 7 months ago |
222-58790 7 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 |
218-64013 7 months ago |
230-81415 7 months ago |
0-109 1 minute |
| 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 |
216-29881 7 months ago |
216-29883 7 months ago |
87-51692 87 days |
| 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 |
216-2210 7 months ago |
216-2210 7 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 |
216-2199 7 months ago |
216-2199 7 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 |
216-2190 7 months ago |
216-2190 7 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 |
216-2180 7 months ago |
216-2180 7 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 |
216-2169 7 months ago |
216-2169 7 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 |
216-2164 7 months ago |
216-2165 7 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 |
216-2159 7 months ago |
216-2159 7 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 |
216-2119 7 months ago |
216-2145 7 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 |
216-2014 7 months ago |
523-78237 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 |
216-2004 7 months ago |
216-2004 7 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 |
216-1939 7 months ago |
216-1939 7 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 |
216-1848 7 months ago |
216-1848 7 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 |
216-1750 7 months ago |
216-1750 7 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 |
216-1738 7 months ago |
216-1738 7 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 |
216-1732 7 months ago |
216-1732 7 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 |
216-1727 7 months ago |
647-58140 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 |
216-1716 7 months ago |
216-1716 7 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 |
216-1680 7 months ago |
216-1680 7 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 |
216-1646 7 months ago |
216-1646 7 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 |
216-1628 7 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 |
216-1479 7 months ago |
216-1479 7 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 |
216-1292 7 months ago |
216-1292 7 months ago |
0-0 0 seconds |
| 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 |
214-80363 7 months ago |
214-80363 7 months ago |
0-0 0 seconds |
| 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 |
212-37122 6 months ago |
212-37122 6 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 |
211-48446 6 months ago |
211-48448 6 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 |
210-64236 6 months ago |
464-77794 1 year ago |
0-0 0 seconds |
| 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 |
203-69515 6 months ago |
228-53819 7 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 |
202-58021 6 months ago |
202-58023 6 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 |
202-58020 6 months ago |
202-58022 6 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 |
201-64051 6 months ago |
201-64052 6 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 |
200-9055 6 months ago |
200-9056 6 months ago |
0-0 0 seconds |
| 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 |
196-34626 6 months ago |
unknown |
unknown |
| 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 |
186-65707 6 months ago |
572-83124 1 year ago |
0-0 0 seconds |
| 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 |
184-82968 6 months ago |
184-82970 6 months ago |
0-0 0 seconds |
| 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 |
184-60465 6 months ago |
unknown |
unknown |
| 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 |
182-16688 5 months ago |
182-16689 5 months ago |
0-16 16 seconds |
| 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 |
182-16688 5 months ago |
182-16690 5 months ago |
285-26861 285 days |
| 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 |
181-25034 5 months ago |
181-25036 5 months ago |
9-22007 9 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 |
180-8181 5 months ago |
455-27812 1 year ago |
28-21477 28 days |
| 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 |
177-24910 5 months ago |
177-24911 5 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 |
176-30222 5 months ago |
176-30224 5 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 |
174-17587 5 months ago |
293-81949 9 months ago |
27-65384 27 days |
| 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 |
168-67649 5 months ago |
168-67651 5 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 |
168-67647 5 months ago |
168-67649 5 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 |
168-67646 5 months ago |
168-67647 5 months ago |
0-638 10 minutes |
| 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 |
165-49937 5 months ago |
403-76153 1 year ago |
129-57991 129 days |
| 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 |
153-17734 5 months ago |
153-17735 5 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 |
153-15512 5 months ago |
153-15513 5 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 |
153-15511 5 months ago |
153-15511 5 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 |
153-15510 5 months ago |
153-15510 5 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 |
153-15509 5 months ago |
153-15509 5 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 |
153-15386 5 months ago |
153-15386 5 months ago |
0-0 0 seconds |
| 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 |
152-52615 4 months ago |
152-52616 4 months ago |
73-67280 73 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 |
148-69826 4 months ago |
148-69828 4 months ago |
179-12934 179 days |
| 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 |
128-62634 4 months ago |
128-62635 4 months ago |
4-80741 4 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 |
126-72950 4 months ago |
126-72950 4 months ago |
0-0 0 seconds |
| 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 |
126-72888 4 months ago |
126-72888 4 months 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 |
126-72797 4 months ago |
126-72797 4 months ago |
0-0 0 seconds |
| 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 |
126-55774 4 months ago |
126-55775 4 months ago |
0-21 21 seconds |
| 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 |
122-79039 4 months ago |
122-79039 4 months 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 |
122-79035 4 months ago |
122-79035 4 months 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 |
122-79026 4 months ago |
122-79026 4 months ago |
2-10495 2 days |
| 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 |
121-81107 3 months ago |
121-81107 3 months 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 |
121-81100 3 months ago |
121-81100 3 months 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 |
121-81094 3 months ago |
121-81094 3 months 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 |
121-81069 3 months ago |
121-81069 3 months 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 |
121-81061 3 months ago |
121-81061 3 months 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 |
121-81053 3 months ago |
121-81053 3 months ago |
0-0 0 seconds |
| 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 |
121-81001 3 months ago |
121-81001 3 months ago |
172-57747 172 days |
| 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 |
121-80837 3 months ago |
121-80837 3 months 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 |
121-80830 3 months ago |
121-80830 3 months ago |
193-70524 193 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 |
121-25381 3 months ago |
121-25382 3 months ago |
0-530 8 minutes |
| 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 |
120-30839 3 months ago |
120-30839 3 months ago |
0-0 0 seconds |
| 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 |
116-77608 3 months ago |
116-77609 3 months ago |
0-0 0 seconds |
| 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 |
113-44760 3 months ago |
113-44761 3 months ago |
0-0 0 seconds |
| 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 |
111-81899 3 months ago |
112-5255 3 months ago |
22-16933 22 days |
| 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 |
108-85153 3 months ago |
108-85154 3 months ago |
0-12793 3 hours |
| 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 |
107-74585 3 months ago |
113-67370 3 months ago |
0-0 0 seconds |
| 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 |
105-22876 3 months ago |
134-57834 4 months ago |
0-0 0 seconds |
| 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 |
104-70261 3 months ago |
233-85266 7 months ago |
52-31623 52 days |
| 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 |
99-32779 3 months ago |
99-32780 3 months ago |
181-72917 181 days |
| 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 |
85-34413 2 months ago |
85-34414 2 months 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
merge-conflict
WIP
|
237/0 |
Mathlib/CategoryTheory/Limits/Skeleton.lean |
1 |
3 |
['alreadydone', 'eric-wieser', 'mathlib4-merge-conflict-bot'] |
nobody |
78-39054 2 months ago |
78-39055 2 months ago |
0-0 0 seconds |
| 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
merge-conflict
awaiting-author
|
76/0 |
Mathlib/Combinatorics/SimpleGraph/Metric.lean |
1 |
3 |
['github-actions', 'leanprover-community-mathlib4-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
67-66002 2 months ago |
67-66003 2 months ago |
1-68738 1 day |
| 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
merge-conflict
awaiting-author
|
376/6 |
Mathlib.lean,Mathlib/Geometry/Manifold/Instances/Real.lean,Mathlib/Geometry/Manifold/Orientable.lean |
3 |
40 |
['Rida-Hamadani', 'github-actions', 'grunweg', 'mathlib4-merge-conflict-bot', 'ocfnash'] |
nobody |
57-62578 1 month ago |
57-62579 1 month ago |
5-70530 5 days |
| 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
merge-conflict
awaiting-author
|
286/1 |
Mathlib.lean,Mathlib/Analysis/SpecialFunctions/Gamma/Beta.lean,Mathlib/Probability/Distributions/Beta.lean |
3 |
50 |
['EtienneC30', 'arulandu', 'github-actions', 'mathlib4-merge-conflict-bot', 'vihdzp'] |
arulandu assignee:arulandu |
55-54384 1 month ago |
57-66854 1 month ago |
1-21124 1 day |
| 9273 |
grunweg author:grunweg |
feat: extended charts are local diffeomorphisms on their source |
---
XXX: is this PR worth keeping, given [isInvertible_mfderiv_extChartAt?](https://leanprover-community.github.io/mathlib4_docs/find/?pattern=isInvertible_mfderiv_extChartAt%3F#doc) shows that extended charts have invertible differential (regardless of whether they are an interior point)?
Perhaps, all one should add is "the differential as an isomorphism..."
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
awaiting-author
|
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 |
52-83542 1 month ago |
unknown |
unknown |
| 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 |
13 |
['Command-Master', 'PatrickMassot', 'dwrensha', 'eric-wieser', 'github-actions', 'grhkm21', 'grunweg', 'kbuzzard', 'kim-em'] |
nobody |
51-40218 1 month ago |
331-84933 10 months ago |
0-8789 2 hours |
| 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 |
48-974 1 month ago |
293-63206 9 months ago |
3-64280 3 days |
| 16428 |
astrainfinita author:astrainfinita |
test use `QuotLike` APIs |
---
- [ ] depends on: #16421
[](https://gitpod.io/from-referrer/)
|
t-data
merge-conflict
|
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', 'mathlib4-dependent-issues-bot'] |
nobody |
47-9338 1 month ago |
47-9340 1 month ago |
0-0 0 seconds |
| 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
merge-conflict
awaiting-author
|
1/1 |
Mathlib/Tactic/GeneralizeProofs.lean |
1 |
5 |
['github-actions', 'jcommelin', 'kmill', 'mathlib4-merge-conflict-bot'] |
nobody |
25-40683 25 days ago |
25-40684 25 days ago |
10-36842 10 days |
| 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
- [x] 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'] |
nobody |
24-43865 24 days ago |
154-56908 5 months ago |
1-33784 1 day |
| 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
merge-conflict
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', 'Vierkantor', 'github-actions', 'grunweg', 'kmill', 'leanprover-bot', 'mathlib4-merge-conflict-bot', 'thorimur', 'urkud'] |
nobody |
18-33381 18 days ago |
unknown |
unknown |
| 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 |
27 |
['TpmKranz', 'YaelDillies', 'dupuisf', 'github-actions', 'leanprover-community-bot-assistant', 'meithecatte', 'rudynicolop'] |
nobody |
17-35209 17 days ago |
199-57768 6 months ago |
45-84611 45 days |
| 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
merge-conflict
WIP
label:t-algebra$ |
86/0 |
Mathlib.lean,Mathlib/LinearAlgebra/Matrix/LinearProgramming.lean |
2 |
15 |
['apurvanakade', 'github-actions', 'leanprover-community-mathlib4-bot', 'madvorak', 'mathlib4-merge-conflict-bot'] |
nobody |
16-68955 16 days ago |
16-68956 16 days 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
merge-conflict
awaiting-author
|
298/0 |
Mathlib.lean,Mathlib/Computability/GNFA.lean,Mathlib/Computability/Language.lean,Mathlib/Computability/RegularExpressions.lean,docs/references.bib |
5 |
7 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'meithecatte', 'trivial1711'] |
nobody |
16-51450 16 days ago |
16-51451 16 days ago |
23-54870 23 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
merge-conflict
awaiting-author
|
159/0 |
Mathlib/Computability/DFA.lean,Mathlib/Computability/Language.lean |
2 |
60 |
['EtienneC30', 'YaelDillies', 'github-actions', 'maemre', 'mathlib4-merge-conflict-bot', 'meithecatte', 'urkud'] |
EtienneC30 assignee:EtienneC30 |
16-50540 16 days ago |
16-50541 16 days ago |
48-67492 48 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
merge-conflict
|
205/0 |
Mathlib.lean,Mathlib/Lean/Meta/AppBuilder.lean |
2 |
1 |
['mathlib4-merge-conflict-bot'] |
nobody |
16-2910 16 days ago |
16-2911 16 days 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
merge-conflict
awaiting-author
|
41/0 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Consume.lean,test/consume.lean |
4 |
5 |
['alexjbest', 'digama0', 'kim-em', 'kmill', 'mathlib4-merge-conflict-bot'] |
nobody |
16-2909 16 days ago |
16-2910 16 days ago |
51-33797 51 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
merge-conflict
WIP
help-wanted
|
287/0 |
Mathlib.lean,Mathlib/Analysis/InnerProductSpace/AffineSubspace.lean |
2 |
7 |
['MithicSpirit', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-merge-conflict-bot'] |
MithicSpirit assignee:MithicSpirit |
16-2907 16 days ago |
16-2907 16 days ago |
0-0 0 seconds |
| 7219 |
Ruben-VandeVelde author:Ruben-VandeVelde |
feat: Equivs for AddMonoidAlgebras |
---
Extracted from #6718.
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
awaiting-author
label:t-algebra$ |
113/0 |
Mathlib.lean,Mathlib/Algebra/MonoidAlgebra/Equiv.lean |
2 |
13 |
['Ruben-VandeVelde', 'alreadydone', 'eric-wieser', 'mathlib4-merge-conflict-bot'] |
eric-wieser assignee:eric-wieser |
16-2905 16 days ago |
16-2906 16 days 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
merge-conflict
WIP
label:t-algebra$ |
87/0 |
Mathlib.lean,Mathlib/LinearAlgebra/LinearProgramming.lean |
2 |
64 |
['Shreyas4991', 'YaelDillies', 'eric-wieser', 'github-actions', 'kim-em', 'madvorak', 'mathlib4-merge-conflict-bot'] |
nobody |
16-2904 16 days ago |
16-2905 16 days ago |
66-6720 66 days |
| 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
merge-conflict
|
141/0 |
Mathlib.lean,Mathlib/Tactic/Common.lean,Mathlib/Tactic/Setm.lean,test/Setm.lean |
4 |
4 |
['mathlib4-merge-conflict-bot', 'thorimur'] |
nobody |
16-2903 16 days ago |
16-2904 16 days 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
merge-conflict
awaiting-author
|
404/0 |
Mathlib.lean,Mathlib/Analysis/Calculus/Gradient/Lemmas.lean |
2 |
31 |
['chenyili0818', 'github-actions', 'jcommelin', 'mathlib4-merge-conflict-bot', 'sgouezel', 'winstonyin'] |
nobody |
16-2779 16 days ago |
16-2780 16 days ago |
51-80670 51 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
merge-conflict
awaiting-author
|
74/0 |
Mathlib.lean,Mathlib/Data/Fiber.lean |
2 |
18 |
['adri326', 'joelriou', 'mathlib4-merge-conflict-bot', 'sinhp'] |
nobody |
16-2778 16 days ago |
16-2779 16 days ago |
1-32924 1 day |
| 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
merge-conflict
awaiting-author
WIP
label:t-algebra$ |
573/0 |
Mathlib.lean,Mathlib/LinearAlgebra/CliffordAlgebra/Basis.lean |
2 |
16 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
16-2774 16 days ago |
16-2775 16 days ago |
0-0 0 seconds |
| 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
merge-conflict
awaiting-author
|
150/0 |
Mathlib.lean,Mathlib/Geometry/Manifold/Algebra/SmoothGerm.lean |
2 |
34 |
['YaelDillies', 'github-actions', 'grunweg', 'jcommelin', 'kim-em', 'mathlib4-merge-conflict-bot', 'mcdoll'] |
fpvandoorn assignee:fpvandoorn |
16-2773 16 days ago |
16-2774 16 days ago |
144-63944 144 days |
| 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
merge-conflict
awaiting-author
|
364/0 |
Mathlib.lean,Mathlib/Logic/Godel/PartArith.lean |
2 |
4 |
['Ruben-VandeVelde', 'YaelDillies', 'mathlib4-merge-conflict-bot'] |
nobody |
16-2772 16 days ago |
16-2773 16 days ago |
97-20483 97 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
merge-conflict
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 |
33 |
['Ruben-VandeVelde', 'eric-wieser', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'smorel394'] |
nobody |
16-2771 16 days ago |
16-2772 16 days ago |
6-23591 6 days |
| 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
merge-conflict
awaiting-author
|
77/0 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter/TerminalRefineLinter.lean |
3 |
15 |
['adomani', 'github-actions', 'grunweg', 'joneugster', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'mathlib4-merge-conflict-bot', 'urkud'] |
nobody |
16-2648 16 days ago |
16-2648 16 days ago |
18-13508 18 days |
| 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/)
|
merge-conflict
WIP
|
152/0 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/SyntaxDataLinter.lean |
3 |
1 |
['mathlib4-merge-conflict-bot'] |
nobody |
16-2647 16 days ago |
16-2647 16 days ago |
0-0 0 seconds |
| 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
merge-conflict
awaiting-author
|
161/0 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Suffa.lean,test/Suffa.lean |
4 |
4 |
['MoritzBeroRoos', 'YaelDillies', 'mathlib4-merge-conflict-bot'] |
nobody |
16-2645 16 days ago |
16-2646 16 days ago |
58-85902 58 days |
| 12632 |
urkud author:urkud |
feat(List/OffDiag): new file |
---
[](https://gitpod.io/from-referrer/)
|
t-data
merge-conflict
awaiting-author
|
221/108 |
Mathlib.lean,Mathlib/Algebra/BigOperators/Group/List/Basic.lean,Mathlib/Data/List/Basic.lean,Mathlib/Data/List/Count.lean,Mathlib/Data/List/Enum.lean,Mathlib/Data/List/Flatten.lean,Mathlib/Data/List/InsertIdx.lean,Mathlib/Data/List/Lattice.lean,Mathlib/Data/List/MinMax.lean,Mathlib/Data/List/NatAntidiagonal.lean,Mathlib/Data/List/Nodup.lean,Mathlib/Data/List/OffDiag.lean,Mathlib/Data/List/Perm/Basic.lean,Mathlib/Data/List/Perm/Lattice.lean,Mathlib/Tactic/GCongr/CoreAttrs.lean |
15 |
4 |
['eric-wieser', 'github-actions', 'mathlib4-merge-conflict-bot', 'urkud'] |
nobody |
16-2644 16 days ago |
16-2645 16 days 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
merge-conflict
modifies-tactic-syntax
awaiting-author
help-wanted
|
439/0 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/MAbel.lean,MathlibTest/mabel.lean |
4 |
11 |
['BoltonBailey', 'dignissimus', 'github-actions', 'joneugster', 'kbuzzard', 'mathlib4-merge-conflict-bot'] |
joneugster assignee:joneugster |
16-2643 16 days ago |
16-2644 16 days ago |
0-16 16 seconds |
| 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
merge-conflict
awaiting-author
label:t-algebra$ |
230/0 |
Mathlib.lean,Mathlib/RingTheory/FractionalIdeal/LocalizedAtPrime.lean,Mathlib/RingTheory/Localization/Basic.lean |
3 |
22 |
['Vierkantor', 'YaelDillies', 'github-actions', 'js2357', 'kbuzzard', 'leanprover-community-bot-assistant', 'leanprover-community-mathlib4-bot', 'mathlib4-merge-conflict-bot'] |
Vierkantor assignee:Vierkantor |
16-2641 16 days ago |
16-2642 16 days ago |
26-39463 26 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
merge-conflict
awaiting-author
|
252/0 |
Mathlib.lean,Mathlib/CategoryTheory/Dialectica/Closed.lean |
2 |
4 |
['github-actions', 'kim-em', 'leanprover-community-mathlib4-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
16-2518 16 days ago |
16-2519 16 days ago |
12-17890 12 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
merge-conflict
awaiting-author
|
37/1 |
Mathlib/RingTheory/Flat/CategoryTheory.lean |
1 |
4 |
['github-actions', 'kim-em', 'mathlib4-merge-conflict-bot'] |
nobody |
16-2516 16 days ago |
16-2516 16 days ago |
3-28223 3 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
merge-conflict
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 |
3 |
['github-actions', 'kim-em', 'mathlib4-merge-conflict-bot'] |
nobody |
16-2514 16 days ago |
16-2515 16 days ago |
6-6256 6 days |
| 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
merge-conflict
awaiting-author
|
185/0 |
Mathlib.lean,Mathlib/CategoryTheory/ConcreteCategory/Pointed.lean,Mathlib/CategoryTheory/Elements.lean |
3 |
14 |
['dagurtomas', 'github-actions', 'kim-em', 'mathlib4-merge-conflict-bot'] |
nobody |
16-2513 16 days ago |
16-2514 16 days ago |
7-80557 7 days |
| 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
merge-conflict
awaiting-author
|
112/0 |
Mathlib.lean,Mathlib/CategoryTheory/Sites/CoveringFamilies.lean |
2 |
21 |
['AnthonyBordg', 'adamtopaz', 'dagurtomas', 'github-actions', 'joelriou', 'mathlib4-merge-conflict-bot'] |
nobody |
16-2512 16 days ago |
16-2513 16 days 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/)
|
merge-conflict |
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 |
5 |
['joneugster', 'mathlib4-merge-conflict-bot', 'mergify'] |
nobody |
16-2510 16 days ago |
16-2510 16 days ago |
0-0 0 seconds |
| 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
merge-conflict
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 |
45 |
['Command-Master', 'adomani', 'bryangingechen', 'edegeltje', 'github-actions', 'grunweg', 'joneugster', 'leanprover-community-bot-assistant', 'mathlib4-merge-conflict-bot'] |
bryangingechen assignee:bryangingechen |
16-2508 16 days ago |
16-2509 16 days ago |
78-54824 78 days |
| 17587 |
kmill author:kmill |
feat: Sym2-as-Finset theory |
---
[](https://gitpod.io/from-referrer/)
|
t-data
new-contributor
merge-conflict
|
105/3 |
Mathlib/Combinatorics/SimpleGraph/Basic.lean,Mathlib/Combinatorics/SimpleGraph/Finite.lean,Mathlib/Data/Sym/Sym2.lean,Mathlib/RingTheory/Polynomial/Vieta.lean |
4 |
11 |
['FordUniver', 'YaelDillies', 'github-actions', 'kmill', 'mathlib4-merge-conflict-bot'] |
nobody |
16-2358 16 days ago |
16-2359 16 days 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
awaiting-CI
merge-conflict
awaiting-author
WIP
label:t-algebra$ |
180/0 |
Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Presheaf/FunctorOfNatTrans.lean |
2 |
6 |
['github-actions', 'kim-em', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
16-2357 16 days ago |
16-2358 16 days ago |
0-0 0 seconds |
| 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
merge-conflict
|
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 |
9 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
16-2356 16 days ago |
16-2356 16 days ago |
0-0 0 seconds |
| 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
merge-conflict
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 |
10 |
['GabinKolly', 'YaelDillies', 'github-actions', 'mathlib4-merge-conflict-bot', 'vihdzp'] |
nobody |
16-2354 16 days ago |
16-2355 16 days ago |
73-63475 73 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
merge-conflict
WIP
|
50/0 |
Mathlib.lean,Mathlib/Data/Sum/Decompose.lean |
2 |
3 |
['github-actions', 'madvorak', 'mathlib4-merge-conflict-bot'] |
nobody |
16-2351 16 days ago |
16-2352 16 days ago |
43-18005 43 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
merge-conflict
awaiting-author
|
101/0 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Widget/Explain.lean |
3 |
9 |
['adamtopaz', 'eric-wieser', 'github-actions', 'joneugster', 'kmill', 'mathlib4-merge-conflict-bot'] |
nobody |
16-2350 16 days ago |
16-2351 16 days ago |
49-80804 49 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
merge-conflict
WIP
|
362/0 |
Mathlib.lean,Mathlib/Data/Finsupp/MonomialOrder/DegLex.lean,Mathlib/Data/Finsupp/MonomialOrder/DegRevLex.lean |
3 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
16-2349 16 days ago |
16-2349 16 days ago |
0-1720 28 minutes |
| 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
merge-conflict
|
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 |
9 |
['eric-wieser', 'github-actions', 'leanprover-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
16-2222 16 days ago |
16-2223 16 days ago |
0-0 0 seconds |
| 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
merge-conflict
awaiting-author
WIP
label:t-algebra$ |
120/0 |
Mathlib.lean,Mathlib/FieldTheory/SimpleExtension.lean |
2 |
19 |
['Command-Master', 'acmepjz', 'github-actions', 'leanprover-community-mathlib4-bot', 'mathlib4-merge-conflict-bot', 'tb65536'] |
nobody |
15-83502 15 days ago |
16-2517 16 days ago |
0-0 0 seconds |
| 6268 |
eric-wieser author:eric-wieser |
fix: 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 |
15-60628 15 days ago |
718-31928 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 |
15-60615 15 days ago |
513-67166 1 year ago |
102-21189 102 days |
| 7427 |
MohanadAhmed author:MohanadAhmed |
feat: eigenvalues sorted in ascending/descending order |
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 |
15-60583 15 days ago |
669-26759 1 year ago |
0-0 0 seconds |
| 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 |
15-60568 15 days ago |
121-80994 3 months ago |
0-0 0 seconds |
| 9564 |
AntoineChambert-Loir author:AntoineChambert-Loir |
chore: 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 |
15-60562 15 days ago |
513-67166 1 year ago |
16-24540 16 days |
| 10026 |
madvorak author:madvorak |
feat: 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
merge-conflict
WIP
label:t-algebra$ |
86/0 |
Mathlib.lean,Mathlib/LinearAlgebra/LinearProgramming.lean |
2 |
10 |
['eric-wieser', 'madvorak', 'mathlib4-merge-conflict-bot', 'riccardobrasca'] |
nobody |
15-60556 15 days ago |
16-2778 16 days ago |
0-0 0 seconds |
| 10159 |
madvorak author:madvorak |
feat: 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
merge-conflict
WIP
label:t-algebra$ |
83/0 |
Mathlib.lean,Mathlib/LinearAlgebra/LinearProgramming.lean |
2 |
8 |
['eric-wieser', 'madvorak', 'mathlib4-merge-conflict-bot', 'riccardobrasca'] |
nobody |
15-60549 15 days ago |
16-2777 16 days ago |
0-0 0 seconds |
| 10349 |
Shamrock-Frost author:Shamrock-Frost |
refactor(CategoryTheory/MorphismProperty): some clean-ups |
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
- [x] 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 |
15-60526 15 days ago |
513-67166 1 year ago |
0-418 6 minutes |
| 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 |
15-60518 15 days ago |
126-72932 4 months ago |
1-20125 1 day |
| 11800 |
JADekker author:JADekker |
feat: 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 |
15-60484 15 days ago |
445-34209 1 year ago |
119-10687 119 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 |
15-60469 15 days ago |
121-81008 3 months ago |
10-75677 10 days |
| 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 |
15-60462 15 days ago |
unknown |
unknown |
| 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 |
15-60457 15 days ago |
282-60136 9 months ago |
2-604 2 days |
| 14426 |
adomani author:adomani |
feat: `#min_imps` command (development branch) |
---
[](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 |
15-60424 15 days ago |
504-82850 1 year ago |
0-0 0 seconds |
| 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 |
15-60413 15 days ago |
304-2086 10 months ago |
0-201 3 minutes |
| 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 |
15-60378 15 days ago |
360-4970 11 months ago |
20-56416 20 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 |
15-60365 15 days ago |
278-57880 9 months ago |
15-40648 15 days |
| 20029 |
FrederickPu author:FrederickPu |
feat(Tactic/simps): 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 |
15-60302 15 days ago |
132-41774 4 months ago |
0-34081 9 hours |
| 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
|
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', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
3-38836 3 days ago |
3-38838 3 days ago |
9-2320 9 days |
| 8224 |
Kha author:Kha |
chore: add `lean4checker` benchmark |
|
merge-conflict
WIP
|
16/0 |
scripts/bench/temci-config.run.yml |
1 |
4 |
['Kha', 'grunweg', 'kim-em', 'leanprover-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
2-40959 2 days ago |
2-40959 2 days ago |
0-0 0 seconds |
| 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 |
325-62275 10 months ago |
325-62275 10 months ago |
6-66637 6 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 |
322-84239 10 months ago |
322-84239 10 months ago |
0-0 0 seconds |
| 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 |
309-42025 10 months ago |
309-42025 10 months ago |
0-9411 2 hours |
| 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 |
297-66763 9 months ago |
298-55126 9 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 |
297-66762 9 months ago |
298-55082 9 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 |
297-66761 9 months ago |
298-54963 9 months ago* |
0-0 0 seconds* |
| 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 |
286-40770 9 months ago |
286-52824 9 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 |
286-39959 9 months ago |
288-73443 9 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 |
285-48643 9 months ago |
286-52387 9 months ago* |
0-0 0 seconds* |
| 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 |
282-139 9 months ago |
282-139 9 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 |
281-61272 9 months ago |
298-55336 9 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 |
281-59636 9 months ago |
298-55200 9 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 |
276-68260 9 months ago |
276-68260 9 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 |
276-68259 9 months ago |
276-68259 9 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 |
276-63094 9 months ago |
276-63094 9 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 |
274-59583 8 months ago |
274-59583 8 months ago |
16-76141 16 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 |
272-60515 8 months ago |
272-60515 8 months ago |
0-0 0 seconds |
| 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 |
266-60181 8 months ago |
266-60181 8 months ago |
1-79072 1 day |
| 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 |
262-81838 8 months ago |
262-81838 8 months ago |
10-48025 10 days |
| 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 |
261-33078 8 months ago |
261-33080 8 months ago |
0-0 0 seconds |
| 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 |
259-38053 8 months ago |
259-38053 8 months ago |
0-0 0 seconds |
| 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 |
257-68296 8 months ago |
257-68296 8 months ago |
0-15573 4 hours |
| 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 |
249-25039 8 months ago |
249-25039 8 months ago |
22-82622 22 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 |
248-14645 8 months ago |
248-14645 8 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 |
248-4408 8 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 |
247-30238 8 months ago |
247-30238 8 months ago |
0-3019 50 minutes |
| 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 |
246-74044 8 months ago |
304-56997 10 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 |
246-66700 8 months ago |
246-66728 8 months ago |
0-84180 23 hours |
| 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 |
245-13431 8 months ago |
245-13432 8 months ago |
0-73190 20 hours |
| 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 |
243-39717 7 months ago |
243-39717 7 months ago |
10-50342 10 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 |
242-35352 7 months ago |
242-35352 7 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 |
242-3657 7 months ago |
242-3658 7 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 |
240-82066 7 months ago |
241-15235 7 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 |
240-6300 7 months ago |
240-6302 7 months ago |
12-18679 12 days |
| 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 |
239-71717 7 months ago |
239-71719 7 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 |
239-67985 7 months ago |
239-67986 7 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 |
239-67983 7 months ago |
239-67985 7 months ago |
43-83249 43 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 |
238-70713 7 months ago |
238-70713 7 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 |
238-4322 7 months ago |
238-7845 7 months ago |
0-568 9 minutes |
| 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 |
233-76602 7 months ago |
233-76604 7 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 |
233-66297 7 months ago |
233-66299 7 months ago |
0-0 0 seconds |
| 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 |
231-41945 7 months ago |
231-41945 7 months ago |
1-17369 1 day |
| 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 |
231-41740 7 months ago |
231-41740 7 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 |
231-40589 7 months ago |
231-40589 7 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 |
231-38043 7 months ago |
231-38043 7 months ago |
13-60072 13 days |
| 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 |
226-80859 7 months ago |
226-80862 7 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 |
224-57634 7 months ago |
224-57636 7 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 |
224-46331 7 months ago |
224-46332 7 months ago |
2-12022 2 days |
| 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 |
222-56506 7 months ago |
263-15199 8 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 |
221-39644 7 months ago |
221-39645 7 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 |
221-39122 7 months ago |
221-39124 7 months ago |
2-7052 2 days |
| 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 |
220-73702 7 months ago |
220-73704 7 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 |
220-66106 7 months ago |
220-66108 7 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 |
219-58774 7 months ago |
219-58776 7 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 |
219-50735 7 months ago |
219-50736 7 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 |
219-11655 7 months ago |
225-77061 7 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 |
219-1073 7 months ago |
219-1075 7 months ago |
0-0 0 seconds |
| 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 |
218-62476 7 months ago |
218-62478 7 months ago |
0-0 0 seconds |
| 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 |
216-17442 7 months ago |
216-17444 7 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 |
216-2658 7 months ago |
216-2658 7 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 |
216-2397 7 months ago |
216-2397 7 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 |
214-62863 7 months ago |
214-62864 7 months ago |
26-25420 26 days |
| 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 |
206-57121 6 months ago |
206-57124 6 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 |
205-78805 6 months ago |
216-2439 7 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 |
205-73180 6 months ago |
216-2434 7 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 |
205-57510 6 months ago |
205-57512 6 months ago |
0-0 0 seconds |
| 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 |
193-65863 6 months ago |
193-65865 6 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 |
193-65344 6 months ago |
193-65345 6 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 |
193-65219 6 months ago |
193-65221 6 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 |
192-71351 6 months ago |
192-71354 6 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 |
192-16668 6 months ago |
192-16669 6 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 |
191-53081 6 months ago |
191-53083 6 months ago |
35-30364 35 days |
| 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 |
184-81829 6 months ago |
184-81830 6 months ago |
64-19141 64 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 |
183-66190 6 months ago |
183-66193 6 months ago |
32-65400 32 days |
| 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 |
182-8167 5 months ago |
182-8168 5 months ago |
0-0 0 seconds |
| 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 |
180-76723 5 months ago |
180-76725 5 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 |
180-75908 5 months ago |
180-75910 5 months ago |
6-40169 6 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 |
180-6175 5 months ago |
180-6177 5 months ago |
0-6023 1 hour |
| 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 |
171-59067 5 months ago |
171-59069 5 months ago |
0-0 0 seconds |
| 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 |
156-65762 5 months ago |
unknown |
unknown |
| 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 |
153-15004 5 months ago |
153-15005 5 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 |
153-15003 5 months ago |
153-15004 5 months ago |
0-0 0 seconds |
| 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 |
153-14996 5 months ago |
153-14996 5 months ago |
82-7297 82 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 |
153-14602 5 months ago |
153-14603 5 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 |
153-14601 5 months ago |
153-14601 5 months ago |
0-0 0 seconds |
| 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 |
153-14598 5 months ago |
153-14598 5 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 |
153-14597 5 months ago |
153-14597 5 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 |
153-14351 5 months ago |
153-14352 5 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 |
153-14349 5 months ago |
153-14350 5 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 |
153-14348 5 months ago |
153-14349 5 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 |
153-14345 5 months ago |
153-14346 5 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 |
153-14344 5 months ago |
153-14344 5 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 |
153-14333 5 months ago |
153-14334 5 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 |
153-14332 5 months ago |
153-14333 5 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 |
153-14206 5 months ago |
153-14207 5 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 |
153-14204 5 months ago |
153-14205 5 months ago |
0-0 0 seconds |
| 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 |
153-14041 5 months ago |
153-14042 5 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 |
153-14039 5 months ago |
153-14039 5 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 |
153-14037 5 months ago |
153-14038 5 months ago |
0-0 0 seconds |
| 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 |
153-12049 5 months ago |
153-12050 5 months ago |
16-56825 16 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 |
151-65868 4 months ago |
151-65869 4 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 |
151-17629 4 months ago |
151-17630 4 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 |
149-81817 4 months ago |
149-81817 4 months ago |
20-8582 20 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 |
148-1491 4 months ago |
149-81819 4 months ago |
21-20473 21 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 |
146-53312 4 months ago |
146-53313 4 months ago |
0-1343 22 minutes |
| 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 |
146-44519 4 months ago |
146-44519 4 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 |
146-23224 4 months ago |
146-52248 4 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 |
144-45376 4 months ago |
144-45377 4 months 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 |
142-70635 4 months ago |
142-70636 4 months ago |
36-35321 36 days |
| 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 |
135-35175 4 months ago |
135-35175 4 months 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 |
134-78461 4 months ago |
134-78463 4 months ago |
0-10930 3 hours |
| 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 |
134-50722 4 months ago |
134-50723 4 months ago |
0-0 0 seconds |
| 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 |
133-81073 4 months ago |
133-81074 4 months ago |
0-0 0 seconds |
| 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 |
132-45092 4 months ago |
132-45093 4 months ago |
23-63406 23 days |
| 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 |
126-72723 4 months 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 |
126-72694 4 months ago |
126-72694 4 months 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 |
126-72559 4 months ago |
126-72559 4 months ago |
0-0 0 seconds |
| 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 |
126-70531 4 months ago |
153-14051 5 months ago |
1-77289 1 day |
| 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 |
126-25346 4 months ago |
126-25347 4 months 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 |
126-25335 4 months ago |
126-25336 4 months 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 |
125-60211 4 months ago |
125-60212 4 months 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 |
125-59977 4 months ago |
127-6056 4 months ago |
37-45446 37 days |
| 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 |
122-79439 4 months ago |
122-79439 4 months ago |
0-0 0 seconds |
| 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 |
122-79321 4 months 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 |
122-79309 4 months ago |
122-79309 4 months 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 |
122-79305 4 months ago |
122-79305 4 months 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 |
122-79300 4 months ago |
122-79300 4 months 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 |
122-79295 4 months ago |
122-79295 4 months 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 |
122-79289 4 months ago |
122-79289 4 months 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 |
122-79284 4 months ago |
122-79284 4 months 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 |
122-79109 4 months ago |
122-79109 4 months 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 |
122-79098 4 months ago |
122-79098 4 months 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 |
122-79089 4 months ago |
122-79089 4 months 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 |
122-79084 4 months ago |
122-79084 4 months 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 |
122-79079 4 months ago |
122-79079 4 months ago |
38-26044 38 days |
| 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 |
122-57798 4 months ago |
122-57798 4 months 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 |
121-81506 3 months ago |
121-81507 3 months 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 |
121-81166 3 months ago |
121-81166 3 months 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 |
121-81129 3 months ago |
121-81129 3 months 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 |
121-81122 3 months ago |
121-81122 3 months ago |
35-86379 35 days |
| 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 |
121-81038 3 months ago |
121-81038 3 months ago |
2-7106 2 days |
| 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 |
121-78565 3 months ago |
121-78566 3 months ago |
1-36700 1 day |
| 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 |
121-30032 3 months ago |
121-30032 3 months ago |
46-52210 46 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 |
121-16185 3 months ago |
121-16185 3 months 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 |
121-14740 3 months ago |
121-14741 3 months 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 |
121-12951 3 months ago |
121-12951 3 months ago |
0-9 9 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 |
120-30561 3 months ago |
120-30562 3 months ago |
0-0 0 seconds |
| 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 |
116-84641 3 months ago |
116-84641 3 months ago |
9-59130 9 days |
| 27451 |
kckennylau author:kckennylau |
feat(RingTheory/Valuation): define ball, closed ball, and sphere |
*From the 2025 Local Class Field Theory Workshop.*
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
merge-conflict
|
27/0 |
Mathlib/RingTheory/Valuation/Basic.lean |
1 |
13 |
['JovanGerb', 'github-actions', 'kckennylau', 'mathlib4-merge-conflict-bot', 'pechersky', 'wwylele'] |
nobody |
115-62535 3 months ago |
115-62536 3 months 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 |
115-62164 3 months ago |
115-62165 3 months 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 |
115-55885 3 months ago |
115-55886 3 months ago |
0-1 1 second |
| 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 |
114-69435 3 months ago |
114-70140 3 months 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 |
113-77324 3 months ago |
113-77325 3 months 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 |
113-76788 3 months ago |
113-76789 3 months ago |
32-70098 32 days |
| 25483 |
VTrelat author:VTrelat |
chore(Data/Set/Prod, SetTheory/ZFC/Basic): add theorem prod_subset_of_prod and extend ZFC model |
Required by @eric-wieser in #24281
---
[](https://gitpod.io/from-referrer/)
|
t-data
new-contributor
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 |
113-66431 3 months ago |
153-14338 5 months ago |
29-56208 29 days |
| 25401 |
digama0 author:digama0 |
feat(Util): SuppressSorry option |
See also leanprover/lean4#8611 and [#lean4 > Silent sorry @ 💬](https://leanprover.zulipchat.com/#narrow/channel/270676-lean4/topic/Silent.20sorry/near/503537964). This is a stop-gap solution while leanprover/lean4#8611 is underway, but it works about as well as any other built in option. Hooking declaration elaborators turns out to be a very powerful technique.
---
[](https://gitpod.io/from-referrer/)
|
t-meta
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 |
113-31584 3 months ago |
113-31584 3 months 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 |
113-31145 3 months ago |
113-31146 3 months ago |
0-70 1 minute |
| 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 |
111-84430 3 months ago |
111-84431 3 months ago |
14-59974 14 days |
| 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 |
110-83979 3 months ago |
110-83980 3 months 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 |
110-74325 3 months ago |
111-2813 3 months 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 |
110-65839 3 months ago |
110-65840 3 months ago |
0-172 2 minutes |
| 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 |
107-35064 3 months ago |
107-35065 3 months 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 |
107-30703 3 months ago |
107-30704 3 months 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 |
106-54927 3 months ago |
106-54928 3 months 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 |
106-48875 3 months ago |
106-62548 3 months 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 |
106-11245 3 months ago |
106-11245 3 months 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 |
105-64190 3 months ago |
105-64191 3 months ago |
2-48353 2 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 |
104-31507 3 months ago |
104-31508 3 months 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 |
104-31506 3 months ago |
104-31507 3 months ago |
13-49738 13 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 |
104-14700 3 months ago |
104-14701 3 months 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 |
104-10826 3 months ago |
126-73148 4 months 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 |
104-10780 3 months ago |
104-10780 3 months ago |
7-4998 7 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 |
103-59058 3 months ago |
126-73149 4 months 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 |
102-62894 3 months ago |
113-30651 3 months 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 |
102-47351 3 months ago |
102-47352 3 months ago |
70-58775 70 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 |
99-61639 3 months ago |
99-61640 3 months ago |
14-30610 14 days |
| 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 |
99-16121 3 months ago |
99-16122 3 months 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 |
99-15992 3 months ago |
99-15993 3 months ago |
16-54453 16 days |
| 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 |
98-14688 3 months ago |
98-14689 3 months ago |
0-0 0 seconds |
| 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 |
97-34526 3 months 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 |
97-34525 3 months ago |
97-34526 3 months 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 |
96-34044 3 months ago |
96-34046 3 months ago |
0-0 0 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 |
94-77498 3 months ago |
94-77499 3 months ago |
19-77946 19 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 |
94-12465 3 months ago |
94-12465 3 months ago |
0-600 10 minutes |
| 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 |
93-29993 3 months ago |
93-29994 3 months ago |
0-20585 5 hours |
| 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 |
93-15681 3 months ago |
93-15682 3 months 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 |
93-12405 3 months ago |
93-13088 3 months ago |
45-34308 45 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 |
90-9111 2 months ago |
90-9112 2 months ago |
40-32085 40 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 |
87-82056 2 months ago |
87-82057 2 months ago |
9-70671 9 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 |
87-62338 2 months ago |
87-62339 2 months 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 |
87-57377 2 months ago |
87-58165 2 months ago |
0-1002 16 minutes |
| 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 |
86-71228 2 months ago |
87-58162 2 months 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 |
86-65213 2 months ago |
86-65214 2 months 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 |
86-65089 2 months ago |
86-65090 2 months ago |
21-3001 21 days |
| 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 |
85-18055 2 months ago |
85-18056 2 months ago |
4-31215 4 days |
| 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 |
84-33074 2 months ago |
84-74963 2 months 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 |
83-38396 2 months ago |
266-3606 8 months ago |
0-27 27 seconds |
| 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 |
83-15722 2 months ago |
83-15723 2 months ago |
39-69478 39 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
merge-conflict
|
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 |
12 |
['Vierkantor', 'github-actions', 'grunweg', 'mathlib4-merge-conflict-bot'] |
nobody |
82-64380 2 months ago |
82-64381 2 months ago |
0-260 4 minutes |
| 29633 |
sgouezel author:sgouezel |
Just for bench |
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict |
1046/690 |
.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/Normed/Module/Basic.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 |
103 |
1 |
['sgouezel'] |
nobody |
81-86364 2 months ago |
82-16 2 months ago* |
0-0 0 seconds* |
| 25069 |
erdOne author:erdOne |
feat(EllipticCurve): rational points of singular nodal cubics |
---
[](https://gitpod.io/from-referrer/)
|
t-algebraic-geometry
merge-conflict
awaiting-author
|
251/0 |
Mathlib.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Affine/Basic.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Singular/Node.lean |
3 |
14 |
['Multramate', 'acmepjz', 'chrisflav', 'erdOne', 'github-actions', 'grunweg', 'mathlib4-merge-conflict-bot'] |
chrisflav assignee:chrisflav |
81-53597 2 months ago |
81-53597 2 months ago |
100-22151 100 days |
| 25070 |
erdOne author:erdOne |
feat(EllipticCurve): rational points on singular cuspidal cubics |
---
[](https://gitpod.io/from-referrer/)
|
t-algebraic-geometry
merge-conflict
awaiting-author
|
123/0 |
Mathlib.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Singular/Cusp.lean |
2 |
12 |
['Multramate', 'acmepjz', 'adamtopaz', 'erdOne', 'github-actions', 'kckennylau', 'mathlib4-merge-conflict-bot'] |
adamtopaz assignee:adamtopaz |
81-53596 2 months ago |
81-53596 2 months ago |
90-52970 90 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
awaiting-author
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 |
80-81890 2 months ago |
80-81890 2 months ago |
49-15167 49 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
merge-conflict
|
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 |
3 |
['ADedecker', 'github-actions', 'mathlib4-merge-conflict-bot'] |
PatrickMassot assignee:PatrickMassot |
80-77333 2 months ago |
80-77334 2 months ago |
87-79752 87 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
merge-conflict
awaiting-author
|
279/11 |
Mathlib.lean,Mathlib/Analysis/InnerProductSpace/GramSchmidtOrtho.lean,Mathlib/Topology/VectorBundle/GramSchmidtOrtho.lean,scripts/noshake.json |
4 |
71 |
['faenuccio', 'github-actions', 'grunweg', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'sgouezel'] |
sgouezel assignee:sgouezel |
80-67990 2 months ago |
80-67991 2 months ago |
28-73015 28 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
merge-conflict
|
14/16 |
Mathlib/Order/Filter/Defs.lean |
1 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
80-65949 2 months ago |
80-65950 2 months ago |
28-42873 28 days |
| 29605 |
alreadydone author:alreadydone |
experiment(Algebra): unbundle npow/zpow from Monoid/InvDivMonoid |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
awaiting-CI
merge-conflict
label:t-algebra$ |
1527/1020 |
Mathlib/Algebra/AddTorsor/Defs.lean,Mathlib/Algebra/BigOperators/Finsupp/Basic.lean,Mathlib/Algebra/BigOperators/Group/Finset/Basic.lean,Mathlib/Algebra/BigOperators/Group/Finset/Defs.lean,Mathlib/Algebra/BigOperators/Group/Finset/Lemmas.lean,Mathlib/Algebra/BigOperators/Group/Finset/Piecewise.lean,Mathlib/Algebra/BigOperators/Group/List/Basic.lean,Mathlib/Algebra/BigOperators/Group/List/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/Pi.lean,Mathlib/Algebra/BigOperators/Ring/Finset.lean,Mathlib/Algebra/BigOperators/Ring/List.lean,Mathlib/Algebra/BigOperators/Ring/Multiset.lean,Mathlib/Algebra/Category/MonCat/ForgetCorepresentable.lean,Mathlib/Algebra/Divisibility/Basic.lean,Mathlib/Algebra/Divisibility/Units.lean,Mathlib/Algebra/Field/Basic.lean,Mathlib/Algebra/Field/Power.lean,Mathlib/Algebra/Field/Rat.lean,Mathlib/Algebra/Group/Action/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/Commute/Units.lean,Mathlib/Algebra/Group/Conj.lean,Mathlib/Algebra/Group/Defs.lean,Mathlib/Algebra/Group/End.lean,Mathlib/Algebra/Group/Even.lean,Mathlib/Algebra/Group/Ext.lean,Mathlib/Algebra/Group/Fin/Basic.lean,Mathlib/Algebra/Group/Finsupp.lean,Mathlib/Algebra/Group/Hom/Basic.lean,Mathlib/Algebra/Group/Hom/Defs.lean,Mathlib/Algebra/Group/Hom/End.lean,Mathlib/Algebra/Group/Hom/Instances.lean,Mathlib/Algebra/Group/Idempotent.lean,Mathlib/Algebra/Group/InjSurj.lean,Mathlib/Algebra/Group/Int/Defs.lean,Mathlib/Algebra/Group/Invertible/Basic.lean,Mathlib/Algebra/Group/Irreducible/Lemmas.lean,Mathlib/Algebra/Group/Nat/Defs.lean,Mathlib/Algebra/Group/Nat/Hom.lean,Mathlib/Algebra/Group/NatPowAssoc.lean,Mathlib/Algebra/Group/Opposite.lean,Mathlib/Algebra/Group/PUnit.lean,Mathlib/Algebra/Group/Pi/Basic.lean,Mathlib/Algebra/Group/Pi/Lemmas.lean,Mathlib/Algebra/Group/Pointwise/Finset/Basic.lean,Mathlib/Algebra/Group/Pointwise/Set/Basic.lean,Mathlib/Algebra/Group/Prod.lean,Mathlib/Algebra/Group/Semiconj/Basic.lean,Mathlib/Algebra/Group/Semiconj/Defs.lean,Mathlib/Algebra/Group/Semiconj/Units.lean,Mathlib/Algebra/Group/Subgroup/Defs.lean,Mathlib/Algebra/Group/Subgroup/Lattice.lean,Mathlib/Algebra/Group/Subgroup/ZPowers/Basic.lean,Mathlib/Algebra/Group/Submonoid/BigOperators.lean,Mathlib/Algebra/Group/Submonoid/Defs.lean,Mathlib/Algebra/Group/Submonoid/Membership.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/Group/Units/Hom.lean,Mathlib/Algebra/GroupWithZero/Action/Defs.lean,Mathlib/Algebra/GroupWithZero/Basic.lean,Mathlib/Algebra/GroupWithZero/Commute.lean,Mathlib/Algebra/GroupWithZero/Conj.lean,Mathlib/Algebra/GroupWithZero/Defs.lean,Mathlib/Algebra/GroupWithZero/Divisibility.lean,Mathlib/Algebra/GroupWithZero/Hom.lean,Mathlib/Algebra/GroupWithZero/Indicator.lean,Mathlib/Algebra/GroupWithZero/InjSurj.lean,Mathlib/Algebra/GroupWithZero/Semiconj.lean,Mathlib/Algebra/GroupWithZero/ULift.lean,Mathlib/Algebra/GroupWithZero/Units/Basic.lean,Mathlib/Algebra/GroupWithZero/Units/Lemmas.lean,Mathlib/Algebra/GroupWithZero/WithZero.lean,Mathlib/Algebra/Module/NatInt.lean,Mathlib/Algebra/NoZeroSMulDivisors/Defs.lean,Mathlib/Algebra/Order/AddGroupWithTop.lean,Mathlib/Algebra/Order/BigOperators/Group/List.lean,Mathlib/Algebra/Order/BigOperators/Group/Multiset.lean,Mathlib/Algebra/Order/BigOperators/GroupWithZero/List.lean,Mathlib/Algebra/Order/BigOperators/GroupWithZero/Multiset.lean,Mathlib/Algebra/Order/Group/Abs.lean,Mathlib/Algebra/Order/Group/Action.lean,Mathlib/Algebra/Order/Group/Basic.lean,Mathlib/Algebra/Order/Group/DenselyOrdered.lean,Mathlib/Algebra/Order/Group/Finset.lean,Mathlib/Algebra/Order/Group/Lattice.lean,Mathlib/Algebra/Order/Group/Multiset.lean,Mathlib/Algebra/Order/Group/PosPart.lean,Mathlib/Algebra/Order/Group/Synonym.lean,Mathlib/Algebra/Order/Group/Unbundled/Abs.lean |
162 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
80-56584 2 months ago |
80-56585 2 months ago |
0-2 2 seconds |
| 29614 |
sgouezel author:sgouezel |
Sg test4 |
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict |
2788/3328 |
.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/ContinuousLinearMap.lean,Mathlib/Analysis/CStarAlgebra/ContinuousMap.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 |
251 |
1 |
['sgouezel'] |
nobody |
79-67511 2 months ago |
82-86153 2 months ago* |
0-0 0 seconds* |
| 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
merge-conflict
|
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 |
10 |
['JovanGerb', 'eric-wieser', 'github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
79-64228 2 months ago |
79-64229 2 months ago |
0-0 0 seconds |
| 29741 |
JovanGerb author:JovanGerb |
trying #28803 using lean#10178 |
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict |
1111/718 |
.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/CStarMatrix.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Instances.lean,Mathlib/Analysis/Normed/Group/Basic.lean,Mathlib/Analysis/Normed/Group/Continuity.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 |
105 |
n/a |
['JovanGerb', 'leanprover-bot'] |
nobody |
78-76135 2 months ago |
unknown |
unknown |
| 29750 |
sgouezel author:sgouezel |
Branch just before the class_abbrev core PR, just for benching |
Branch just before the class_abbrev core PR, just for benching
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict |
1041/684 |
.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/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,lean-toolchain |
101 |
1 |
['sgouezel'] |
nobody |
78-62737 2 months ago |
78-62796 2 months ago* |
0-0 0 seconds* |
| 25138 |
chrisflav author:chrisflav |
chore(RingTheory/Ideal): make `RingHom.ker` take a `RingHom` instead of `RingHomClass` |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
label:t-algebra$ |
105/95 |
Mathlib/Algebra/Algebra/Hom.lean,Mathlib/Algebra/Algebra/Subalgebra/Operations.lean,Mathlib/Algebra/Category/CommAlgCat/FiniteType.lean,Mathlib/Algebra/Polynomial/Module/AEval.lean,Mathlib/Combinatorics/Nullstellensatz.lean,Mathlib/FieldTheory/Minpoly/Field.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,Mathlib/Topology/ContinuousMap/StoneWeierstrass.lean |
18 |
6 |
['chrisflav', 'erdOne', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-merge-conflict-bot'] |
nobody |
77-56482 2 months ago |
77-56483 2 months ago |
16-338 16 days |
| 27972 |
smmercuri author:smmercuri |
refactor: 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
WIP
label:t-algebra$ |
186/93 |
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 |
7 |
['github-actions', 'leanprover-bot', 'mathlib4-merge-conflict-bot', 'smmercuri'] |
nobody |
74-32943 2 months ago |
74-32944 2 months ago |
3-83441 3 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
merge-conflict
awaiting-author
|
103/0 |
Mathlib.lean,Mathlib/CategoryTheory/Limits/Types/OverPullback.lean,Mathlib/CategoryTheory/Limits/Types/Shapes.lean |
3 |
10 |
['emilyriehl', 'github-actions', 'joelriou', 'mathlib4-merge-conflict-bot', 'robin-carlier', 'sinhp'] |
nobody |
73-48619 2 months ago |
73-48619 2 months ago |
13-55990 13 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
merge-conflict
WIP
label:t-algebra$ |
120/15 |
Mathlib/LinearAlgebra/RootSystem/Defs.lean,Mathlib/LinearAlgebra/RootSystem/Finite/G2.lean,Mathlib/LinearAlgebra/RootSystem/Reduced.lean |
3 |
9 |
['eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'ocfnash'] |
nobody |
72-4419 2 months ago |
72-4420 2 months ago |
0-1 1 second |
| 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
merge-conflict
|
61/68 |
Mathlib/GroupTheory/Perm/Fin.lean |
1 |
10 |
['JovanGerb', 'eric-wieser', 'github-actions', 'mathlib4-merge-conflict-bot', 'plp127', 'tb65536'] |
nobody |
72-2530 2 months ago |
72-2531 2 months ago |
20-39203 20 days |
| 29829 |
vihdzp author:vihdzp |
draft: more stuff on `standardPart` |
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict |
549/10 |
Mathlib.lean,Mathlib/Algebra/Order/Archimedean/Class.lean,Mathlib/Algebra/Order/Archimedean/Hom.lean,Mathlib/Algebra/Order/CompleteField.lean,Mathlib/Algebra/Order/Ring/Archimedean.lean,Mathlib/Data/Real/StandardPart.lean,Mathlib/Order/Quotient.lean |
7 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
71-85370 2 months ago |
71-85371 2 months ago |
0-0 0 seconds |
| 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
merge-conflict
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 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
71-12788 2 months ago |
71-12789 2 months ago |
0-0 0 seconds |
| 29657 |
jcreinhold author:jcreinhold |
feat(CategoryTheory/MarkovCategory): add Markov categories |
This PR adds Markov categories to the category theory library. A Markov category is a symmetric monoidal category where every object has canonical copy and delete morphisms that form commutative comonoids.
## What this gives mathlib
In a Markov category, morphisms model probabilistic processes. The copy morphism `X → X ⊗ X` creates perfect correlation (both outputs always equal). The delete morphism `X → I` marginalizes (sums/integrates out variables).
This structure captures probability theory categorically. The same theorem proves results for:
- Finite probability (stochastic matrices)
- Measure theory (Markov kernels)
- Kleisli categories of probability monads
Fritz (2020) used this to prove categorical versions of Fisher-Neyman, Basu's theorem, and other core statistics results.
## Implementation
- `MarkovCategory`: Extends `SymmetricCategory` with canonical comonoid structure
- `copyMor X : X ⟶ X ⊗ X` and `delMor X : X ⟶ I` for each object
- Coherence axioms: commutativity, counitality, coassociativity
- Compatibility with tensor products
Key design point: The comonoid structure is canonical (fields of the typeclass), not chosen. This matches the probability interpretation where there's exactly one way to copy/marginalize.
## Examples included
1. Cartesian categories: Every cartesian monoidal category forms a Markov category where copy is the diagonal `x ↦ (x,x)` and delete is the terminal morphism. All morphisms are deterministic.
2. FinStoch: Objects are finite types. Morphisms are stochastic matrices (rows sum to 1). This models finite probability spaces with the usual matrix multiplication for composition.
## Scope and review notes
This PR provides the basic structure only. Future PRs would add:
- Conditional independence
- Sufficient statistics
- Connection to measure-theoretic probability
- More examples (Kleisli categories, Gaussian categories)
I'm neither an expert in this material nor in Lean; I've only read a few papers on Markov categories and have gone through tutorial material in Lean. Please review for mathematical correctness and idiomatic Lean. I kept this PR small to check if mathlib wants this addition and to ensure it meets repository standards.
## Why add this now
Markov categories provide a useful abstraction level for probability in type theory. Adding it to mathlib enables future work on categorical probability and statistics. In particular, I'm working on a probabilistic programming library and would like to write some proofs using these constructs.
## References
- Fritz, T. (2020). [A synthetic approach to Markov kernels, conditional independence and theorems on sufficient statistics](https://arxiv.org/abs/1908.07021). *Advances in Mathematics*, 370, 107239.
- Cho, K., & Jacobs, B. (2019). [Disintegration and Bayesian inversion via string diagrams](https://arxiv.org/abs/1709.00322). *Mathematical Structures in Computer Science*, 29(7), 938-971.
---
All definitions include docstrings. The PR has tests for the core functionality.
[](https://gitpod.io/from-referrer/) |
new-contributor
t-category-theory
merge-conflict
awaiting-author
|
2414/7 |
Mathlib.lean,Mathlib/CategoryTheory/Bicategory/Monad/Basic.lean,Mathlib/CategoryTheory/CopyDiscardCategory/Basic.lean,Mathlib/CategoryTheory/CopyDiscardCategory/Deterministic.lean,Mathlib/CategoryTheory/MarkovCategory/Basic.lean,Mathlib/CategoryTheory/MarkovCategory/Cartesian.lean,Mathlib/CategoryTheory/MarkovCategory/FinStoch/Basic.lean,Mathlib/CategoryTheory/MarkovCategory/FinStoch/Braided.lean,Mathlib/CategoryTheory/MarkovCategory/FinStoch/CopyDiscard.lean,Mathlib/CategoryTheory/MarkovCategory/FinStoch/Markov.lean,Mathlib/CategoryTheory/MarkovCategory/FinStoch/Monoidal.lean,Mathlib/CategoryTheory/Monoidal/Bimon_.lean,Mathlib/CategoryTheory/Monoidal/CommComon_.lean,Mathlib/CategoryTheory/Monoidal/Comon_.lean,MathlibTest/CategoryTheory/MarkovCategory.lean,docs/references.bib |
16 |
28 |
['github-actions', 'jcreinhold', 'joelriou', 'mathlib4-merge-conflict-bot'] |
nobody |
70-65120 2 months ago |
70-65121 2 months ago |
0-0 0 seconds |
| 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
|
235/237 |
.gitignore,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 |
22 |
9 |
['github-actions', 'harahu', 'mathlib4-merge-conflict-bot'] |
nobody |
70-19325 2 months ago |
70-19326 2 months ago |
0-0 0 seconds |
| 27829 |
dupuisf author:dupuisf |
feat: modify `cfc_tac` to use `grind` |
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict
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 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
69-67031 2 months ago |
69-67032 2 months ago |
0-1 1 second |
| 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 |
33 |
['Ruben-VandeVelde', 'erdOne', 'faenuccio', 'github-actions', 'leanprover-community-bot-assistant', 'pechersky', 'smmercuri', 'xroblot'] |
nobody |
69-64040 2 months ago |
150-63977 4 months ago |
79-1228 79 days |
| 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
merge-conflict
|
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 |
70 |
['IvanRenison', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'themathqueen'] |
themathqueen assignee:themathqueen |
68-65870 2 months ago |
68-65871 2 months ago |
2-57966 2 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
merge-conflict
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 |
6 |
['Ruben-VandeVelde', 'fpvandoorn', 'github-actions', 'grunweg', 'mathlib4-merge-conflict-bot'] |
nobody |
67-37188 2 months ago |
67-37189 2 months ago |
0-24361 6 hours |
| 21035 |
mattrobball author:mattrobball |
draft |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
label:t-algebra$ |
3/3 |
Mathlib/RingTheory/Kaehler/JacobiZariski.lean |
1 |
5 |
['github-actions', 'leanprover-bot', 'mathlib4-merge-conflict-bot', 'mattrobball'] |
nobody |
66-79498 2 months ago |
66-79498 2 months ago |
0-0 0 seconds |
| 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 |
6 |
['chrisflav', 'github-actions', 'leanprover-community-bot-assistant', 'ppls-nd-prs', 'robin-carlier'] |
nobody |
66-79333 2 months ago |
153-12039 5 months ago |
0-47665 13 hours |
| 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
merge-conflict
|
786/1 |
Mathlib.lean,Mathlib/CategoryTheory/Limits/Shapes/Pullback/Categorical/Basic.lean,Mathlib/CategoryTheory/Limits/Shapes/Pullback/Categorical/Square.lean |
3 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
66-54122 2 months ago |
66-54123 2 months ago |
0-5521 1 hour |
| 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
merge-conflict
label:t-algebra$ |
54/42 |
Mathlib/Algebra/Module/Submodule/Defs.lean |
1 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
66-17156 2 months ago |
66-17156 2 months ago |
0-0 0 seconds |
| 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
|
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 |
65-73524 2 months ago |
65-73526 2 months ago |
0-1708 28 minutes |
| 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/)
|
merge-conflict
WIP
|
64/0 |
Mathlib/Analysis/Normed/Module/FiniteDimension.lean,Mathlib/LinearAlgebra/BilinearMap.lean |
2 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
65-39891 2 months ago |
65-39892 2 months ago |
0-2 2 seconds |
| 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
- [x] depends on: #26547
[](https://gitpod.io/from-referrer/)
|
large-import
t-category-theory
merge-conflict
|
205/0 |
Mathlib/CategoryTheory/Limits/Shapes/Pullback/Categorical/CatCospanTransform.lean |
1 |
5 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
64-76749 2 months ago |
64-79721 2 months ago |
0-625 10 minutes |
| 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
merge-conflict
|
148/2 |
Mathlib/Topology/FiberBundle/Trivialization.lean,Mathlib/Topology/Maps/Basic.lean |
2 |
4 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
ADedecker assignee:ADedecker |
63-79193 2 months ago |
63-79194 2 months ago |
134-68375 134 days |
| 26115 |
grunweg author:grunweg |
WIP/proof of concept,feat: the inverse function theorem for manifolds |
---
[](https://gitpod.io/from-referrer/)
|
t-differential-geometry
merge-conflict
WIP
|
348/0 |
Mathlib.lean,Mathlib/Analysis/Calculus/ContDiff/Defs.lean,Mathlib/Geometry/Manifold/InverseFunctionTheorem.lean,Mathlib/Topology/PartialHomeomorph.lean |
4 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
63-78636 2 months ago |
63-78637 2 months ago |
0-0 0 seconds |
| 29012 |
grunweg author:grunweg |
chore: reduce `Topology` imports in `Data` |
Move Data.Real.Sqrt to Analysis.
---
- [ ] depends on: #28966
[](https://gitpod.io/from-referrer/)
|
file-removed
merge-conflict
|
25/21 |
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/Normed/Module/Ball/Homeomorph.lean,Mathlib/Analysis/RCLike/Basic.lean,Mathlib/Analysis/Real/Sqrt.lean,Mathlib/Data/Rat/NatSqrt/Real.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 |
20 |
5 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
62-72062 2 months ago |
62-72063 2 months ago |
6-26396 6 days |
| 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
merge-conflict
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 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-merge-conflict-bot'] |
nobody |
62-59863 2 months ago |
62-59864 2 months ago |
0-10 10 seconds |
| 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 |
['YaelDillies', 'astrainfinita', 'github-actions', 'grunweg', 'leanprover-bot', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
kbuzzard assignee:kbuzzard |
61-58464 2 months ago |
unknown |
unknown |
| 30192 |
erdOne author:erdOne |
feat(RingTheory): valuative topology = adic topology for discrete rank 1 valuations |
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
t-topology
merge-conflict
WIP
|
190/2 |
Mathlib.lean,Mathlib/Order/Filter/Bases/Basic.lean,Mathlib/RingTheory/Valuation/ValuativeRel/Basic.lean,Mathlib/RingTheory/Valuation/ValuativeRel/Integers.lean,Mathlib/Topology/Algebra/Nonarchimedean/AdicTopology.lean,Mathlib/Topology/Algebra/Valued/ValuativeRel.lean |
6 |
3 |
['erdOne', 'github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
60-74187 1 month ago |
60-74187 1 month ago |
0-331 5 minutes |
| 26344 |
mans0954 author:mans0954 |
feat(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 |
60-52772 1 month ago |
123-81054 4 months ago |
5-43696 5 days |
| 25992 |
Multramate author:Multramate |
feat(RingTheory/Ideal/Span): add pair lemmas |
This PR continues the work from #25323.
Original PR: https://github.com/leanprover-community/mathlib4/pull/25323 |
t-ring-theory
merge-conflict
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 |
10 |
['Multramate', 'Ruben-VandeVelde', 'github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
59-49733 1 month ago |
59-49735 1 month ago |
39-76045 39 days |
| 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/)
|
merge-conflict |
259/14 |
Mathlib/Algebra/Group/Submonoid/Defs.lean,Mathlib/GroupTheory/Finiteness.lean |
2 |
4 |
['github-actions', 'mathlib4-merge-conflict-bot', 'plp127', 'uniwuni'] |
dupuisf assignee:dupuisf |
57-80393 1 month ago |
57-80394 1 month ago |
25-78230 25 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` |
merge-conflict
awaiting-author
|
191/0 |
Mathlib/Analysis/InnerProductSpace/Orthogonal.lean |
1 |
8 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'sgouezel', 'yoh-tanimoto'] |
sgouezel assignee:sgouezel |
57-65125 1 month ago |
57-65126 1 month ago |
12-74361 12 days |
| 29926 |
jcreinhold author:jcreinhold |
feat(CategoryTheory/MarkovCategory): add basic finite stochastic matrices definitions to Markov category |
This PR introduces FinStoch, the category of finite stochastic matrices, as a concrete example of a Markov category.
This PR builds on #29925, #29939, and #29919 and was split up from #29657.
## Main additions
### 1. Core definitions (`FinStoch/Basic.lean`)
- `StochasticMatrix m n`: Matrices where rows sum to 1, representing conditional probabilities P(j|i)
- `FinStoch`: The category with finite types as objects and stochastic matrices as morphisms
- `DetMorphism`: Deterministic matrices (exactly one 1 per row) with their underlying functions
- Composition: Matrix multiplication preserves row-stochasticity via the Chapman-Kolmogorov equation
Key design choices:
- Row-stochastic convention: entry (i,j) is P(output=j | input=i)
- Deterministic morphisms tracked separately for structural isomorphisms
### 2. Monoidal structure (`FinStoch/Monoidal.lean`)
Implements tensor products modeling independent parallel processes:
- Tensor on objects: Cartesian product of finite types
- Tensor on morphisms: Kronecker product P((j₁,j₂)|(i₁,i₂)) = P(j₁|i₁) × P(j₂|i₂)
- Structural morphisms: Associator, unitors use deterministic permutations
- Coherence**: Pentagon and triangle identities verified computationally
## Mathematical significance
FinStoch provides the canonical example of a Markov category:
- Morphisms: Stochastic matrices/Markov chains
- Composition: Chapman-Kolmogorov equation for multi-step transitions
- Tensor: Independent parallel processes
This models finite probability spaces categorically, where:
- Objects represent sample spaces
- Morphisms represent probabilistic transitions
- Tensor products model independence
## References
Fritz (2020)
- [ ] depends on: #29925 |
new-contributor
t-category-theory
merge-conflict
|
1437/0 |
Mathlib.lean,Mathlib/CategoryTheory/CopyDiscardCategory/Basic.lean,Mathlib/CategoryTheory/CopyDiscardCategory/Deterministic.lean,Mathlib/CategoryTheory/MarkovCategory/Basic.lean,Mathlib/CategoryTheory/MarkovCategory/Cartesian.lean,Mathlib/CategoryTheory/MarkovCategory/FinStoch/Basic.lean,Mathlib/CategoryTheory/MarkovCategory/FinStoch/Monoidal.lean,MathlibTest/CategoryTheory/MarkovCategory.lean,docs/references.bib |
9 |
4 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
55-55534 1 month ago |
55-55536 1 month ago |
0-0 0 seconds |
| 30359 |
JLimperg author:JLimperg |
[Not a PR] Benchmark for Aesop RPINF precompilation |
---
[](https://gitpod.io/from-referrer/)
|
file-removed
merge-conflict
|
5/3 |
lake-manifest.json,lakefile.lean,scripts/bench/fake-root/lib/lean/libleanshared.so,scripts/bench/run |
4 |
5 |
['JLimperg', 'github-actions', 'leanprover-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
55-46391 1 month ago |
55-46392 1 month ago |
0-0 0 seconds |
| 30351 |
JLimperg author:JLimperg |
[Not a PR] Benchmark Aesop's lazy forward state construction |
Testing the performance impact of an Aesop change.
---
[](https://gitpod.io/from-referrer/)
|
dependency-bump
merge-conflict
|
3/3 |
lake-manifest.json,lakefile.lean |
2 |
11 |
['JLimperg', 'github-actions', 'leanprover-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
55-35292 1 month ago |
55-46394 1 month ago |
0-0 0 seconds |
| 30425 |
JLimperg author:JLimperg |
[Not a PR] Benchmark Aesop with precompiled RPINF at instance transparency |
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict |
5/3 |
lake-manifest.json,lakefile.lean,scripts/bench/fake-root/lib/lean/libleanshared.so,scripts/bench/run |
4 |
2 |
['JLimperg', 'leanprover-bot'] |
nobody |
55-28496 1 month ago |
55-30691 1 month ago |
0-0 0 seconds |
| 30438 |
JLimperg author:JLimperg |
[Not a PR] Benchmark Aesop change that computes fewer RPINFs |
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict |
5/3 |
lake-manifest.json,lakefile.lean,scripts/bench/fake-root/lib/lean/libleanshared.so,scripts/bench/run |
4 |
5 |
['JLimperg', 'github-actions', 'leanprover-bot'] |
nobody |
54-58873 1 month ago |
54-64991 1 month ago |
0-0 0 seconds |
| 30440 |
JLimperg author:JLimperg |
[Not a PR] Benchmark Aesop with no `hypTypes` in `ForwardState` and `instances` RPINF transparency |
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict |
5/3 |
lake-manifest.json,lakefile.lean,scripts/bench/fake-root/lib/lean/libleanshared.so,scripts/bench/run |
4 |
3 |
['JLimperg', 'github-actions', 'leanprover-bot'] |
nobody |
54-54354 1 month ago |
54-57072 1 month ago |
0-0 0 seconds |
| 30452 |
JLimperg author:JLimperg |
[Not a PR] Benchmark Aesop with no `hypTypes` in `ForwardState`, RPINF at `instances` transparency and lazy forward state |
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict |
5/3 |
lake-manifest.json,lakefile.lean,scripts/bench/fake-root/lib/lean/libleanshared.so,scripts/bench/run |
4 |
3 |
['JLimperg', 'github-actions', 'leanprover-bot'] |
nobody |
54-35233 1 month ago |
54-37362 1 month ago |
0-0 0 seconds |
| 22657 |
Xmask19 author:Xmask19 |
feat: a graph is maximally acyclic iff it is a tree |
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-combinatorics
merge-conflict
|
86/0 |
Mathlib/Combinatorics/SimpleGraph/Acyclic.lean |
1 |
7 |
['Rida-Hamadani', 'b-mehta', 'github-actions', 'grunweg', 'mathlib4-merge-conflict-bot'] |
b-mehta assignee:b-mehta |
54-34572 1 month ago |
54-34573 1 month ago |
208-19611 208 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
merge-conflict
|
172/0 |
Counterexamples.lean,Counterexamples/DiscreteTopologyWithNontrivialValuation.lean |
2 |
n/a |
['github-actions', 'grunweg', 'kckennylau', 'mathlib4-merge-conflict-bot', 'pechersky'] |
nobody |
53-60595 1 month ago |
unknown |
unknown |
| 24434 |
joelriou author:joelriou |
feat(CategoryTheory): effectiveness of descent |
(This is very much a draft, it will be split in multiple PRs later.)
Co-authored-by: Christian Merten [christian@merten.dev](mailto:christian@merten.dev)
---
- [x] depends on: #24411
- [x] depends on: #24382
- [ ] depends on: #25971
- [x] depends on: #13539
[](https://gitpod.io/from-referrer/)
|
t-category-theory
merge-conflict
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', 'yuma-mizuno'] |
nobody |
53-60571 1 month ago |
unknown |
unknown |
| 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.
---
- [x] depends on: #28242
[](https://gitpod.io/from-referrer/)
|
t-category-theory
merge-conflict
awaiting-author
|
165/23 |
Mathlib.lean,Mathlib/CategoryTheory/Bicategory/EqToHom.lean,Mathlib/CategoryTheory/Bicategory/Strict.lean,Mathlib/CategoryTheory/EqToHom.lean,scripts/noshake.json |
5 |
9 |
['github-actions', 'joelriou', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'robin-carlier'] |
nobody |
53-57333 1 month ago |
61-36018 2 months ago |
0-9063 2 hours |
| 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
merge-conflict
|
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 |
5 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
52-57894 1 month ago |
52-57895 1 month ago |
44-45896 44 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
merge-conflict
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 |
51-30002 1 month ago |
unknown |
unknown |
| 29378 |
mans0954 author:mans0954 |
feat(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
merge-conflict
|
133/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 |
6 |
4 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
51-17031 1 month ago |
51-17032 1 month ago |
0-14664 4 hours |
| 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
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 |
50-67457 1 month ago |
50-67460 1 month ago |
0-0 0 seconds |
| 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
merge-conflict
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 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
50-62171 1 month ago |
50-62172 1 month ago |
0-28 28 seconds |
| 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
merge-conflict
|
0/564 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/LinearCombination'.lean,Mathlib/Tactic/Linter/UnusedTactic.lean,MathlibTest/linear_combination'.lean |
5 |
4 |
['euprunin', 'github-actions', 'grunweg', 'mathlib4-merge-conflict-bot'] |
nobody |
50-7203 1 month ago |
50-7204 1 month ago |
0-1 1 second |
| 28826 |
alreadydone author:alreadydone |
feat(CategoryTheory): Additive and Linear when Hom types are only monoids |
+ 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
WIP
|
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 |
47-81159 1 month ago |
48-37112 1 month ago |
0-1 1 second |
| 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
merge-conflict
awaiting-author
|
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 |
11 |
['Sebi-Kumar', 'alreadydone', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'mattrobball'] |
mattrobball assignee:mattrobball |
47-48716 1 month ago |
47-48717 1 month ago |
14-30316 14 days |
| 30642 |
thorimur author:thorimur |
bench: lean4#10832 |
|
large-import
merge-conflict
|
507/460 |
.github/workflows/nightly-docgen.yml,Cache/IO.lean,Mathlib.lean,Mathlib/Algebra/Algebra/StrictPositivity.lean,Mathlib/Algebra/BigOperators/Group/List/Basic.lean,Mathlib/Algebra/BigOperators/Group/List/Lemmas.lean,Mathlib/Algebra/Group/Units/Defs.lean,Mathlib/Algebra/Notation/Defs.lean,Mathlib/Algebra/Order/Ring/Unbundled/Rat.lean,Mathlib/Algebra/Polynomial/RuleOfSigns.lean,Mathlib/AlgebraicTopology/SimplexCategory/GeneratorsRelations/NormalForms.lean,Mathlib/Analysis/LocallyConvex/WithSeminorms.lean,Mathlib/Analysis/SpecialFunctions/ContinuousFunctionalCalculus/ExpLog.lean,Mathlib/Analysis/SpecialFunctions/ContinuousFunctionalCalculus/Rpow/Basic.lean,Mathlib/Combinatorics/SimpleGraph/CompleteMultipartite.lean,Mathlib/Combinatorics/SimpleGraph/FiveWheelLike.lean,Mathlib/Computability/DFA.lean,Mathlib/Computability/RegularExpressions.lean,Mathlib/Control/Monad/Cont.lean,Mathlib/Data/Finset/Attach.lean,Mathlib/Data/Finset/Defs.lean,Mathlib/Data/Finset/Empty.lean,Mathlib/Data/Finsupp/Notation.lean,Mathlib/Data/Fintype/Defs.lean,Mathlib/Data/Fintype/EquivFin.lean,Mathlib/Data/Int/LeastGreatest.lean,Mathlib/Data/List/Chain.lean,Mathlib/Data/List/Flatten.lean,Mathlib/Data/List/SplitOn.lean,Mathlib/Data/List/Triplewise.lean,Mathlib/Data/Multiset/ZeroCons.lean,Mathlib/Data/Nat/Digits/Defs.lean,Mathlib/Data/Set/Basic.lean,Mathlib/Data/Set/Insert.lean,Mathlib/Data/Set/Operations.lean,Mathlib/Data/String/Basic.lean,Mathlib/Data/String/Defs.lean,Mathlib/Data/String/Lemmas.lean,Mathlib/Lean/Elab/InfoTree.lean,Mathlib/MeasureTheory/Integral/IntervalIntegral/LebesgueDifferentiationThm.lean,Mathlib/Order/CompleteLattice/MulticoequalizerDiagram.lean,Mathlib/SetTheory/PGame/Basic.lean,Mathlib/Tactic/Basic.lean,Mathlib/Tactic/DeclarationNames.lean,Mathlib/Tactic/Hint.lean,Mathlib/Tactic/Linter/CommandStart.lean,Mathlib/Tactic/Linter/DocString.lean,Mathlib/Tactic/Linter/Header.lean,Mathlib/Tactic/Linter/TextBased.lean,Mathlib/Tactic/Says.lean,Mathlib/Tactic/SuccessIfFailWithMsg.lean,Mathlib/Tactic/ToAdditive/Frontend.lean,Mathlib/Tactic/ToAdditive/GuessName.lean,Mathlib/Tactic/ToExpr.lean,Mathlib/Tactic/Widget/Calc.lean,Mathlib/Tactic/Widget/CongrM.lean,Mathlib/Tactic/Widget/Conv.lean,Mathlib/Tactic/Widget/GCongr.lean,Mathlib/Tactic/Widget/InteractiveUnfold.lean,Mathlib/Tactic/Widget/LibraryRewrite.lean,Mathlib/Tactic/Widget/SelectPanelUtils.lean,Mathlib/Util/CompileInductive.lean,Mathlib/Util/Superscript.lean,MathlibTest/CalcQuestionMark.lean,MathlibTest/Change.lean,MathlibTest/DeprecateTo.lean,MathlibTest/FieldSimp.lean,MathlibTest/FindSyntax.lean,MathlibTest/LibraryRewrite.lean,MathlibTest/LibrarySearch/basic.lean,MathlibTest/LibrarySearch/mathlib.lean,MathlibTest/LibrarySearch/observe.lean,MathlibTest/Simps.lean,MathlibTest/Subsingleton.lean,MathlibTest/Use.lean,MathlibTest/Util/PrintSorries.lean,MathlibTest/Variable.lean,MathlibTest/fast_instance.lean,MathlibTest/grind/pairwise_disjoint.lean,MathlibTest/hint.lean,MathlibTest/propose.lean,MathlibTest/rewrites.lean,MathlibTest/ring.lean,MathlibTest/says.lean,MathlibTest/says_whitespace.lean,MathlibTest/success_if_fail_with_msg.lean,MathlibTest/toAdditive.lean,lake-manifest.json,lakefile.lean,lean-toolchain,scripts/check-yaml.lean,scripts/noshake.json |
92 |
4 |
['github-actions', 'leanprover-bot', 'mathlib4-merge-conflict-bot', 'thorimur'] |
nobody |
46-55548 1 month ago |
48-8571 1 month ago* |
0-0 0 seconds* |
| 30643 |
thorimur author:thorimur |
bench: before lean4#10832 |
|
large-import
merge-conflict
|
507/460 |
.github/workflows/nightly-docgen.yml,Cache/IO.lean,Mathlib.lean,Mathlib/Algebra/Algebra/StrictPositivity.lean,Mathlib/Algebra/BigOperators/Group/List/Basic.lean,Mathlib/Algebra/BigOperators/Group/List/Lemmas.lean,Mathlib/Algebra/Group/Units/Defs.lean,Mathlib/Algebra/Notation/Defs.lean,Mathlib/Algebra/Order/Ring/Unbundled/Rat.lean,Mathlib/Algebra/Polynomial/RuleOfSigns.lean,Mathlib/AlgebraicTopology/SimplexCategory/GeneratorsRelations/NormalForms.lean,Mathlib/Analysis/LocallyConvex/WithSeminorms.lean,Mathlib/Analysis/SpecialFunctions/ContinuousFunctionalCalculus/ExpLog.lean,Mathlib/Analysis/SpecialFunctions/ContinuousFunctionalCalculus/Rpow/Basic.lean,Mathlib/Combinatorics/SimpleGraph/CompleteMultipartite.lean,Mathlib/Combinatorics/SimpleGraph/FiveWheelLike.lean,Mathlib/Computability/DFA.lean,Mathlib/Computability/RegularExpressions.lean,Mathlib/Control/Monad/Cont.lean,Mathlib/Data/Finset/Attach.lean,Mathlib/Data/Finset/Defs.lean,Mathlib/Data/Finset/Empty.lean,Mathlib/Data/Finsupp/Notation.lean,Mathlib/Data/Fintype/Defs.lean,Mathlib/Data/Fintype/EquivFin.lean,Mathlib/Data/Int/LeastGreatest.lean,Mathlib/Data/List/Chain.lean,Mathlib/Data/List/Flatten.lean,Mathlib/Data/List/SplitOn.lean,Mathlib/Data/List/Triplewise.lean,Mathlib/Data/Multiset/ZeroCons.lean,Mathlib/Data/Nat/Digits/Defs.lean,Mathlib/Data/Set/Basic.lean,Mathlib/Data/Set/Insert.lean,Mathlib/Data/Set/Operations.lean,Mathlib/Data/String/Basic.lean,Mathlib/Data/String/Defs.lean,Mathlib/Data/String/Lemmas.lean,Mathlib/Lean/Elab/InfoTree.lean,Mathlib/MeasureTheory/Integral/IntervalIntegral/LebesgueDifferentiationThm.lean,Mathlib/Order/CompleteLattice/MulticoequalizerDiagram.lean,Mathlib/SetTheory/PGame/Basic.lean,Mathlib/Tactic/Basic.lean,Mathlib/Tactic/DeclarationNames.lean,Mathlib/Tactic/Hint.lean,Mathlib/Tactic/Linter/CommandStart.lean,Mathlib/Tactic/Linter/DocString.lean,Mathlib/Tactic/Linter/Header.lean,Mathlib/Tactic/Linter/TextBased.lean,Mathlib/Tactic/Says.lean,Mathlib/Tactic/SuccessIfFailWithMsg.lean,Mathlib/Tactic/ToAdditive/Frontend.lean,Mathlib/Tactic/ToAdditive/GuessName.lean,Mathlib/Tactic/ToExpr.lean,Mathlib/Tactic/Widget/Calc.lean,Mathlib/Tactic/Widget/CongrM.lean,Mathlib/Tactic/Widget/Conv.lean,Mathlib/Tactic/Widget/GCongr.lean,Mathlib/Tactic/Widget/InteractiveUnfold.lean,Mathlib/Tactic/Widget/LibraryRewrite.lean,Mathlib/Tactic/Widget/SelectPanelUtils.lean,Mathlib/Util/CompileInductive.lean,Mathlib/Util/Superscript.lean,MathlibTest/CalcQuestionMark.lean,MathlibTest/Change.lean,MathlibTest/DeprecateTo.lean,MathlibTest/FieldSimp.lean,MathlibTest/FindSyntax.lean,MathlibTest/LibraryRewrite.lean,MathlibTest/LibrarySearch/basic.lean,MathlibTest/LibrarySearch/mathlib.lean,MathlibTest/LibrarySearch/observe.lean,MathlibTest/Simps.lean,MathlibTest/Subsingleton.lean,MathlibTest/Use.lean,MathlibTest/Util/PrintSorries.lean,MathlibTest/Variable.lean,MathlibTest/fast_instance.lean,MathlibTest/grind/pairwise_disjoint.lean,MathlibTest/hint.lean,MathlibTest/propose.lean,MathlibTest/rewrites.lean,MathlibTest/ring.lean,MathlibTest/says.lean,MathlibTest/says_whitespace.lean,MathlibTest/success_if_fail_with_msg.lean,MathlibTest/toAdditive.lean,lake-manifest.json,lakefile.lean,lean-toolchain,scripts/check-yaml.lean,scripts/noshake.json |
92 |
4 |
['github-actions', 'leanprover-bot', 'mathlib4-merge-conflict-bot', 'thorimur'] |
nobody |
46-55547 1 month ago |
48-7519 1 month ago* |
0-0 0 seconds* |
| 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
merge-conflict
label:t-algebra$ |
122/5 |
Mathlib/LinearAlgebra/FreeProduct/Basic.lean |
1 |
26 |
['YaelDillies', 'adomani', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'robertmaxton42'] |
nobody |
43-18016 1 month ago |
43-18017 1 month ago |
165-29512 165 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
merge-conflict
|
29/9 |
Mathlib/Data/Set/Basic.lean,Mathlib/Data/Set/Operations.lean |
2 |
5 |
['dupuisf', 'euprunin', 'github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
42-55705 1 month ago |
42-55706 1 month ago |
84-66723 84 days |
| 25978 |
Bergschaf author:Bergschaf |
feat(Order/Sublocale): Open Sublocales |
---
[](https://gitpod.io/from-referrer/)
- [x] 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 |
42-49451 1 month ago |
115-7327 3 months ago |
0-1908 31 minutes |
| 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
merge-conflict
|
158/0 |
Mathlib.lean,Mathlib/Algebra/BigOperators/Ring/Finset.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Bounds.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/SeriesBounds.lean |
4 |
28 |
['Parcly-Taxel', 'Ruben-VandeVelde', 'adomani', 'girving', 'github-actions', 'llllvvuu', 'mathlib4-merge-conflict-bot', 'urkud'] |
nobody |
42-47088 1 month ago |
42-47089 1 month ago |
48-80227 48 days |
| 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/)
|
merge-conflict
awaiting-author
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 |
11 |
['eric-wieser', 'github-actions', 'grunweg', 'mathlib4-merge-conflict-bot', 'thorimur'] |
nobody |
39-81670 1 month ago |
39-81670 1 month ago |
0-61617 17 hours |
| 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/)
|
merge-conflict
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 |
17 |
['b-mehta', 'github-actions', 'leanprover-bot', 'mathlib-bors', 'mathlib4-merge-conflict-bot', 'mattrobball'] |
nobody |
38-55096 1 month ago |
38-55097 1 month ago |
0-5717 1 hour |
| 28737 |
astrainfinita author:astrainfinita |
refactor: deprecate `MulEquivClass` |
This PR continues the work from #18806.
Original PR: https://github.com/leanprover-community/mathlib4/pull/18806 |
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 |
37-84085 1 month ago |
37-84085 1 month ago |
4-17723 4 days |
| 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
merge-conflict
awaiting-author
|
45/5 |
Mathlib/NumberTheory/ArithmeticFunction.lean |
1 |
19 |
['MichaelStollBayreuth', 'SnirBroshi', 'b-mehta', 'eric-wieser', 'github-actions', 'mathlib4-merge-conflict-bot', 'riccardobrasca', 'sun123zxy'] |
MichaelStollBayreuth assignee:MichaelStollBayreuth |
37-84037 1 month ago |
37-84037 1 month ago |
53-41880 53 days |
| 30421 |
grunweg author:grunweg |
WIP: support products in the differential geometry elaborators |
Nothing to see yet. Best reviewed commit by commit.
---
- [ ] depends on: #30413
[](https://gitpod.io/from-referrer/)
|
merge-conflict |
1051/254 |
Mathlib/Geometry/Manifold/Notation.lean,Mathlib/Lean/Meta/Basic.lean,MathlibTest/DifferentialGeometry/Notation.lean,MathlibTest/DifferentialGeometry/NotationAdvanced.lean |
4 |
4 |
['github-actions', 'grunweg', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
37-78689 1 month ago |
37-78691 1 month ago |
0-2190 36 minutes |
| 30299 |
franv314 author:franv314 |
feat(Topology/Instances): Cantor set |
Prove that the Cantor set has empty interior and the cardinality of the continuum as discussed on [Zulip](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/A.20few.20results.20about.20the.20Cantor.20set/with/543560670)
Moves:
- Mathlib.Topology.Instances.CantorSet -> Mathlib.Topology.Instances.CantorSet.Basic
---
[](https://gitpod.io/from-referrer/)
|
file-removed
new-contributor
t-topology
merge-conflict
awaiting-author
|
355/2 |
Mathlib.lean,Mathlib/Topology/Instances/CantorSet/Basic.lean,Mathlib/Topology/Instances/CantorSet/Cardinality.lean,Mathlib/Topology/Instances/CantorSet/Lemmas.lean |
4 |
5 |
['github-actions', 'grunweg', 'kckennylau', 'mathlib4-merge-conflict-bot'] |
nobody |
37-75767 1 month ago |
37-75768 1 month ago |
0-2409 40 minutes |
| 30690 |
grunweg author:grunweg |
style(Order): fix whitespace |
Extracted from #30658. Found by extending the commandStart linter to proof bodies.
---
[](https://gitpod.io/from-referrer/)
|
t-order
merge-conflict
|
69/69 |
Mathlib/Order/Basic.lean,Mathlib/Order/Bounds/Image.lean,Mathlib/Order/Defs/PartialOrder.lean,Mathlib/Order/Filter/Cocardinal.lean,Mathlib/Order/Heyting/Basic.lean,Mathlib/Order/KonigLemma.lean,Mathlib/Order/Max.lean,Mathlib/Order/Minimal.lean,Mathlib/Order/Monotone/Basic.lean,Mathlib/Order/PiLex.lean,Mathlib/Order/RelClasses.lean,Mathlib/Order/SetIsMax.lean,Mathlib/Order/SetNotation.lean,Mathlib/Order/WithBot.lean |
14 |
4 |
['JovanGerb', 'github-actions', 'grunweg', 'mathlib4-merge-conflict-bot'] |
Vierkantor assignee:Vierkantor |
37-74630 1 month ago |
37-74631 1 month ago |
8-67789 8 days |
| 30393 |
mans0954 author:mans0954 |
WIP: Bipolar theorem absconvex refactor |
Experiment to see what happens when #26345 and #29342 are merged.
---
[](https://gitpod.io/from-referrer/)
|
large-import
merge-conflict
WIP
|
383/138 |
Mathlib.lean,Mathlib/Analysis/Convex/Basic.lean,Mathlib/Analysis/LocallyConvex/AbsConvex.lean,Mathlib/Analysis/LocallyConvex/AbsConvexOpen.lean,Mathlib/Analysis/LocallyConvex/Basic.lean,Mathlib/Analysis/LocallyConvex/Bipolar.lean,Mathlib/Analysis/LocallyConvex/Polar.lean,Mathlib/Analysis/LocallyConvex/WeakDual.lean,Mathlib/Analysis/Normed/Module/Dual.lean,Mathlib/Topology/Algebra/Module/LinearSpan.lean,Mathlib/Topology/Algebra/Module/StrongTopology.lean,Mathlib/Topology/Algebra/Module/WeakBilin.lean |
12 |
n/a |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
37-57476 1 month ago |
unknown |
unknown |
| 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
merge-conflict
WIP
|
22/0 |
Mathlib/NumberTheory/NumberField/InfinitePlace/Ramification.lean |
1 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
36-61607 1 month ago |
36-61608 1 month ago |
0-57 57 seconds |
| 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
merge-conflict
awaiting-author
|
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 |
10 |
['adamtopaz', 'github-actions', 'javra', 'mathlib4-merge-conflict-bot'] |
adamtopaz assignee:adamtopaz |
35-20202 1 month ago |
35-20202 1 month ago |
78-31643 78 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
merge-conflict
please-adopt
WIP
|
75/6 |
Mathlib/Geometry/Manifold/Diffeomorph.lean,Mathlib/Geometry/Manifold/LocalDiffeomorph.lean |
2 |
3 |
['github-actions', 'grunweg', 'mathlib4-merge-conflict-bot'] |
nobody |
34-78605 1 month ago |
34-78606 1 month ago |
0-74 1 minute |
| 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
merge-conflict
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 |
32 |
['ADedecker', 'eric-wieser', 'github-actions', 'mathlib-bors', 'mathlib4-merge-conflict-bot', 'ocfnash'] |
ocfnash assignee:ocfnash |
34-67341 1 month ago |
34-67342 1 month ago |
28-12053 28 days |
| 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/)
|
merge-conflict |
2/2 |
Mathlib/Tactic/Linter/Style.lean,Mathlib/Tactic/TacticAnalysis.lean |
2 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
34-63842 1 month ago |
34-63843 1 month ago |
0-0 0 seconds |
| 30790 |
urkud author:urkud |
chore: partially migrate from `ContinuousMap.continuous` |
... to `map_continuous` or `by fun_prop`.
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict |
37/45 |
Mathlib/AlgebraicGeometry/Morphisms/Constructors.lean,Mathlib/AlgebraicTopology/FundamentalGroupoid/Basic.lean,Mathlib/AlgebraicTopology/FundamentalGroupoid/FundamentalGroup.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Restrict.lean,Mathlib/Analysis/Complex/Circle.lean,Mathlib/Analysis/Fourier/AddCircleMulti.lean,Mathlib/Condensed/Light/TopCatAdjunction.lean,Mathlib/Condensed/TopCatAdjunction.lean,Mathlib/Condensed/TopComparison.lean,Mathlib/Dynamics/Ergodic/Action/OfMinimal.lean,Mathlib/MeasureTheory/Constructions/BorelSpace/Basic.lean,Mathlib/Topology/Category/CompHausLike/Limits.lean,Mathlib/Topology/Compactification/OnePoint/Basic.lean,Mathlib/Topology/Compactness/CompactlyGeneratedSpace.lean,Mathlib/Topology/ContinuousMap/CompactlySupported.lean,Mathlib/Topology/ContinuousMap/Units.lean,Mathlib/Topology/ContinuousMap/ZeroAtInfty.lean,Mathlib/Topology/LocallyConstant/Basic.lean,Mathlib/Topology/PartitionOfUnity.lean,Mathlib/Topology/Sets/Opens.lean,Mathlib/Topology/TietzeExtension.lean,Mathlib/Topology/UniformSpace/CompactConvergence.lean,Mathlib/Topology/UniformSpace/Dini.lean,Mathlib/Topology/UrysohnsLemma.lean |
24 |
6 |
['erdOne', 'github-actions', 'mathlib4-merge-conflict-bot', 'urkud'] |
nobody |
34-63145 1 month ago |
34-63146 1 month ago |
8-85332 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
merge-conflict
awaiting-author
|
30/0 |
Mathlib/Topology/LocallyFinsupp.lean |
1 |
22 |
['Raph-DG', 'chrisflav', 'github-actions', 'jcommelin', 'kckennylau', 'mathlib4-merge-conflict-bot', 'urkud'] |
j-loreaux assignee:j-loreaux |
31-71583 1 month ago |
31-71583 1 month ago |
118-44502 118 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
merge-conflict
awaiting-author
|
129/110 |
Mathlib/RingTheory/MatrixAlgebra.lean |
1 |
28 |
['Whysoserioushah', 'chrisflav', 'eric-wieser', 'github-actions', 'jcommelin', 'mathlib-bors', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'mattrobball'] |
chrisflav assignee:chrisflav |
31-62865 1 month ago |
31-62866 1 month ago |
63-50556 63 days |
| 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 |
165/126 |
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/LinearAlgebra/Basis/Defs.lean,Mathlib/LinearAlgebra/Determinant.lean,Mathlib/LinearAlgebra/Finsupp/VectorSpace.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/Rank.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 |
19 |
4 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-merge-conflict-bot'] |
nobody |
31-45266 1 month ago |
31-45268 1 month ago |
62-52011 62 days |
| 29638 |
yuma-mizuno author:yuma-mizuno |
feat(CategoryTheory): define descent data by presieves |
---
Addendum: I realized that there is prior work in #24434. Since this PR uses a slightly different definition, I plan to make this PR a follow-up to #24434. Until then, I’ll keep it marked as WIP. See the comment: https://github.com/leanprover-community/mathlib4/pull/29638#issuecomment-3290041719
[](https://gitpod.io/from-referrer/)
|
t-category-theory
merge-conflict
WIP
|
408/2 |
Mathlib.lean,Mathlib/CategoryTheory/Bicategory/Functor/Pseudofunctor.lean,Mathlib/CategoryTheory/Bicategory/LocallyDiscrete.lean,Mathlib/CategoryTheory/Category/Cat.lean,Mathlib/CategoryTheory/Stack/Basic.lean,Mathlib/CategoryTheory/Stack/Descent.lean |
6 |
7 |
['chrisflav', 'github-actions', 'joelriou', 'mathlib4-merge-conflict-bot', 'yuma-mizuno'] |
nobody |
31-41363 1 month ago |
31-41364 1 month ago |
0-74 1 minute |
| 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/)
|
sphere-packing
large-import
new-contributor
t-analysis
merge-conflict
|
201/0 |
Mathlib/Analysis/Complex/CauchyIntegral.lean |
1 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
31-35302 1 month ago |
31-35303 1 month ago |
0-0 0 seconds |
| 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 |
91 |
['EtienneC30', 'b-mehta', 'ctchou', 'github-actions', 'leanprover-community-bot-assistant', 'meithecatte', 'rudynicolop'] |
EtienneC30 assignee:EtienneC30 |
31-16893 1 month ago |
199-56843 6 months ago |
39-67601 39 days |
| 31220 |
fgdorais author:fgdorais |
chore: adaptations for batteries#1489 |
After [batteries#1489](https://github.com/leanprover-community/batteries/pull/1489) is merged:
- [ ] Edit the lakefile to point to leanprover-community/batteries:main
- [ ] Run lake update batteries
- [ ] Merge leanprover-community/mathlib4:master
- [ ] Wait for CI and merge |
large-import
blocked-by-batt-PR
merge-conflict
|
12/35 |
Mathlib/Data/Array/Extract.lean,lake-manifest.json,lakefile.lean |
3 |
3 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
31-14656 1 month ago |
31-14657 1 month ago |
0-15 15 seconds |
| 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
merge-conflict
awaiting-author
|
58/16 |
Mathlib/SetTheory/ZFC/Basic.lean,Mathlib/SetTheory/ZFC/Ordinal.lean |
2 |
5 |
['alreadydone', 'b-mehta', 'github-actions', 'mathlib4-merge-conflict-bot', 'vihdzp'] |
alreadydone assignee:alreadydone |
30-74021 1 month ago |
30-74022 1 month ago |
12-2927 12 days |
| 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.)
(It would make sense to redefine `CommGrp/Grp/CommMon` as full subcategories of `Mon`, rather than defining `CommGrp` by applying `InducedCategory` twice, which adds one unnecessary layer of `.hom`, but no attempt was made to change this in this PR.)
---
(This time, I will try to complete this refactor. I very much need this for applications to homotopical algebra, where full subcategories of cofibrant/fibrant/bifibrant objects are used.)
[](https://gitpod.io/from-referrer/)
|
large-import
t-category-theory
merge-conflict
WIP
|
2002/1459 |
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/SimplexCategory/Truncated.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 |
142 |
8 |
['erdOne', 'github-actions', 'joelriou', 'leanprover-community-bot-assistant', 'mathlib4-merge-conflict-bot', 'smorel394'] |
nobody |
30-68972 1 month ago |
30-68973 1 month ago |
0-2 2 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
merge-conflict
awaiting-author
|
438/3 |
Mathlib.lean,Mathlib/Algebra/GroupWithZero/Action/Basic.lean,Mathlib/RingTheory/DiscreteValuationRing/Basic.lean,Mathlib/RingTheory/OrderOfVanishing/Basic.lean,Mathlib/RingTheory/OrderOfVanishing/Properties.lean |
5 |
18 |
['Raph-DG', 'erdOne', 'github-actions', 'mathlib4-merge-conflict-bot'] |
erdOne assignee:erdOne |
30-48613 1 month ago |
30-48613 1 month ago |
33-5791 33 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
merge-conflict
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 |
3 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
kim-em assignee:kim-em |
30-37193 1 month ago |
30-37194 1 month ago |
80-71575 80 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
|
624/100 |
Mathlib/Algebra/MvPolynomial/Eval.lean,Mathlib/Algebra/MvPolynomial/Expand.lean,Mathlib/Algebra/Order/Floor/Semifield.lean,Mathlib/Algebra/Order/Positive/Field.lean,Mathlib/Algebra/Order/Positive/Ring.lean,Mathlib/Data/Int/ModEq.lean,Mathlib/Data/NNRat/Floor.lean,Mathlib/Data/Nat/Factorial/Basic.lean,Mathlib/Data/Nat/ModEq.lean,Mathlib/Data/Nat/NthRoot/Defs.lean,Mathlib/Data/Rat/Floor.lean,Mathlib/Tactic/NormNum/Basic.lean,MathlibTest/norm_num_ext.lean |
13 |
4 |
['github-actions', 'grunweg', 'mathlib4-merge-conflict-bot'] |
nobody |
30-4916 1 month ago |
30-4917 1 month ago |
0-0 0 seconds |
| 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. ]
- [x] depends on: #26225
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebraic-geometry
merge-conflict
awaiting-author
|
269/1 |
Mathlib/AlgebraicGeometry/Properties.lean,Mathlib/Order/KrullDimension.lean,Mathlib/Topology/KrullDimension.lean,Mathlib/Topology/Sober.lean |
4 |
37 |
['Raph-DG', 'chrisflav', 'erdOne', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
erdOne assignee:erdOne |
29-78237 29 days ago |
31-59012 1 month ago |
28-60757 28 days |
| 30686 |
grunweg author:grunweg |
tracking: #30658 split into pieces |
---
- [x] depends on: #30685
- [x] depends on: #30687
- [x] depends on: #30688
- [x] depends on: #30689
- [x] depends on: #30762 (revert the other changes)
- [x] depends on: #30691
- [x] depends on: #30778
Not meant for merging, but for me tracking the changes locally. This PR should never land directly.
[](https://gitpod.io/from-referrer/)
|
large-import
merge-conflict
|
2327/245 |
Mathlib/Algebra/AddConstMap/Basic.lean,Mathlib/Algebra/Algebra/Spectrum/Quasispectrum.lean,Mathlib/Algebra/BrauerGroup/Defs.lean,Mathlib/Algebra/Category/Ring/Basic.lean,Mathlib/Algebra/GroupWithZero/Range.lean,Mathlib/Algebra/IsPrimePow.lean,Mathlib/Algebra/MonoidAlgebra/ToDirectSum.lean,Mathlib/Algebra/NoZeroSMulDivisors/Basic.lean,Mathlib/Algebra/Order/CauSeq/Basic.lean,Mathlib/Algebra/Order/Module/Defs.lean,Mathlib/Algebra/Polynomial/AlgebraMap.lean,Mathlib/Algebra/Ring/BooleanRing.lean,Mathlib/Algebra/SkewMonoidAlgebra/Basic.lean,Mathlib/AlgebraicGeometry/AffineSpace.lean,Mathlib/AlgebraicTopology/DoldKan/EquivalencePseudoabelian.lean,Mathlib/AlgebraicTopology/SimplexCategory/GeneratorsRelations/EpiMono.lean,Mathlib/AlgebraicTopology/SimplicialSet/StdSimplex.lean,Mathlib/Analysis/BoxIntegral/UnitPartition.lean,Mathlib/Analysis/Calculus/ContDiff/FTaylorSeries.lean,Mathlib/Analysis/Calculus/ContDiff/FaaDiBruno.lean,Mathlib/Analysis/Complex/UpperHalfPlane/Topology.lean,Mathlib/Analysis/Normed/Unbundled/SmoothingSeminorm.lean,Mathlib/CategoryTheory/Abelian/Projective/Resolution.lean,Mathlib/CategoryTheory/Bicategory/Adjunction/Mate.lean,Mathlib/CategoryTheory/Bicategory/EqToHom.lean,Mathlib/CategoryTheory/Category/Cat/Adjunction.lean,Mathlib/CategoryTheory/Category/Cat/Terminal.lean,Mathlib/CategoryTheory/Closed/Ideal.lean,Mathlib/CategoryTheory/Core.lean,Mathlib/CategoryTheory/Enriched/FunctorCategory.lean,Mathlib/CategoryTheory/EqToHom.lean,Mathlib/CategoryTheory/FiberedCategory/Cartesian.lean,Mathlib/CategoryTheory/FiberedCategory/HomLift.lean,Mathlib/CategoryTheory/Functor/KanExtension/Basic.lean,Mathlib/CategoryTheory/Grothendieck.lean,Mathlib/CategoryTheory/IsConnected.lean,Mathlib/CategoryTheory/Limits/FilteredColimitCommutesFiniteLimit.lean,Mathlib/CategoryTheory/Limits/Presheaf.lean,Mathlib/CategoryTheory/Limits/Shapes/BinaryProducts.lean,Mathlib/CategoryTheory/Limits/Shapes/Pullback/Categorical/Basic.lean,Mathlib/CategoryTheory/Limits/Shapes/Pullback/Categorical/CatCospanTransform.lean,Mathlib/CategoryTheory/Limits/Shapes/Reflexive.lean,Mathlib/CategoryTheory/Limits/Sifted.lean,Mathlib/CategoryTheory/Limits/Types/Colimits.lean,Mathlib/CategoryTheory/Localization/CalculusOfFractions.lean,Mathlib/CategoryTheory/Localization/Monoidal/Braided.lean,Mathlib/CategoryTheory/Monad/Adjunction.lean,Mathlib/CategoryTheory/Monad/Equalizer.lean,Mathlib/CategoryTheory/Monoidal/Action/Basic.lean,Mathlib/CategoryTheory/Monoidal/Action/End.lean,Mathlib/CategoryTheory/Monoidal/DayConvolution/Closed.lean,Mathlib/CategoryTheory/Monoidal/ExternalProduct/Basic.lean,Mathlib/CategoryTheory/Monoidal/Opposite.lean,Mathlib/CategoryTheory/Quotient.lean,Mathlib/CategoryTheory/Shift/Induced.lean,Mathlib/CategoryTheory/Sites/Coherent/SequentialLimit.lean,Mathlib/CategoryTheory/Sites/CoverLifting.lean,Mathlib/CategoryTheory/Sites/Monoidal.lean,Mathlib/CategoryTheory/Subpresheaf/Subobject.lean,Mathlib/CategoryTheory/Yoneda.lean,Mathlib/Combinatorics/Matroid/Closure.lean,Mathlib/Combinatorics/Matroid/Rank/ENat.lean,Mathlib/Data/EReal/Operations.lean,Mathlib/Data/Fin/Fin2.lean,Mathlib/Data/Fin/Tuple/Curry.lean,Mathlib/Data/Fin/Tuple/Embedding.lean,Mathlib/Data/Finset/Card.lean,Mathlib/Data/List/Lemmas.lean,Mathlib/Data/List/Sort.lean,Mathlib/Data/Nat/ChineseRemainder.lean,Mathlib/Data/Nat/Digits/Defs.lean,Mathlib/Data/Nat/MaxPowDiv.lean,Mathlib/Data/Nat/ModEq.lean,Mathlib/Data/Nat/Prime/Defs.lean,Mathlib/Data/Num/Bitwise.lean,Mathlib/Data/Ordmap/Ordset.lean,Mathlib/Data/Real/Basic.lean,Mathlib/Data/Seq/Computation.lean,Mathlib/Data/Set/Insert.lean,Mathlib/Data/Set/Prod.lean,Mathlib/Data/Vector/MapLemmas.lean,Mathlib/FieldTheory/IsSepClosed.lean,Mathlib/Geometry/Manifold/ContMDiffMFDeriv.lean,Mathlib/Geometry/Manifold/Instances/Real.lean,Mathlib/GroupTheory/Coxeter/Inversion.lean,Mathlib/GroupTheory/FreeGroup/Reduce.lean,Mathlib/GroupTheory/GroupAction/Jordan.lean,Mathlib/Lean/Meta/RefinedDiscrTree/Basic.lean,Mathlib/LinearAlgebra/Alternating/Basic.lean,Mathlib/LinearAlgebra/ExteriorPower/Basic.lean,Mathlib/LinearAlgebra/PiTensorProduct.lean,Mathlib/LinearAlgebra/QuadraticForm/Basic.lean,Mathlib/LinearAlgebra/RootSystem/Hom.lean,Mathlib/Logic/Function/FromTypes.lean,Mathlib/MeasureTheory/SetAlgebra.lean,Mathlib/ModelTheory/Fraisse.lean,Mathlib/NumberTheory/Cyclotomic/PrimitiveRoots.lean,Mathlib/NumberTheory/Dioph.lean,Mathlib/NumberTheory/LucasLehmer.lean,Mathlib/NumberTheory/ModularForms/EisensteinSeries/Summable.lean |
128 |
5 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
29-43251 29 days ago |
29-43252 29 days ago |
13-17060 13 days |
| 29877 |
Komyyy author:Komyyy |
feat: inner product of the gradient |
Also, this PR enables the `conj` notation in the file.
---
[](https://gitpod.io/from-referrer/)
|
t-analysis
merge-conflict
|
37/10 |
Mathlib/Analysis/Calculus/Gradient/Basic.lean |
1 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
hrmacbeth assignee:hrmacbeth |
28-65852 28 days ago |
28-65854 28 days ago |
45-5432 45 days |
| 29992 |
vlad902 author:vlad902 |
feat(Order): finite (Max)Chains always contains a top/max element |
---
- [ ] depends on: #29835 [optional extra text]
- [ ] depends on: #29993 [optional extra text]
[](https://gitpod.io/from-referrer/)
|
large-import
t-order
merge-conflict
WIP
|
35/0 |
Mathlib/Order/Preorder/Chain.lean |
1 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
28-56997 28 days ago |
29-48237 29 days ago |
0-466 7 minutes |
| 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
merge-conflict
awaiting-author
|
198/0 |
Mathlib.lean,Mathlib/Tactic/Simproc/PolynomialDegree.lean,MathlibTest/polynomial_degree_simproc.lean |
3 |
19 |
['5hv5hvnk', 'YaelDillies', 'adomani', 'github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
28-55086 28 days ago |
28-55087 28 days ago |
2-71043 2 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
merge-conflict
awaiting-author
|
114/0 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Simproc/Matrix.lean,scripts/noshake.json |
4 |
6 |
['Vierkantor', 'github-actions', 'kckennylau', 'mathlib4-merge-conflict-bot'] |
alexjbest assignee:alexjbest |
28-54840 28 days ago |
28-54841 28 days ago |
58-77127 58 days |
| 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
merge-conflict
WIP
help-wanted
|
249/0 |
Mathlib.lean,Mathlib/Analysis/NormedSpace/HahnBanach/Splits.lean |
2 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
28-41849 28 days ago |
28-41850 28 days ago |
0-0 0 seconds |
| 31020 |
grunweg author:grunweg |
feat: mfderiv of Sum.inl and Sum.inr |
Nothing to see yet: waiting on the cache, then I will state the sorries and Newell Jansen has expressed interest in trying to prove this.
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict
WIP
|
64/0 |
Mathlib/Geometry/Manifold/MFDeriv/SpecificFunctions.lean |
1 |
4 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
28-40614 28 days ago |
28-40615 28 days ago |
0-1 1 second |
| 26345 |
mans0954 author:mans0954 |
feat(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
merge-conflict
awaiting-author
|
334/93 |
Mathlib.lean,Mathlib/Analysis/LocallyConvex/AbsConvex.lean,Mathlib/Analysis/LocallyConvex/Bipolar.lean,Mathlib/Analysis/LocallyConvex/Polar.lean,Mathlib/Analysis/LocallyConvex/WeakDual.lean,Mathlib/Analysis/Normed/Module/Dual.lean,Mathlib/Topology/Algebra/Module/LinearSpan.lean,Mathlib/Topology/Algebra/Module/StrongTopology.lean,Mathlib/Topology/Algebra/Module/WeakBilin.lean |
9 |
n/a |
['JonBannon', 'eric-wieser', 'faenuccio', 'github-actions', 'j-loreaux', 'leanprover-community-bot-assistant', 'mans0954', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'mcdoll'] |
nobody |
28-39254 28 days ago |
unknown |
unknown |
| 30908 |
vihdzp author:vihdzp |
refactor: swap `Function.update_apply` and `Pi.single_apply` |
These are backwards compared to `Finsupp.single_apply`, `DFinsupp.single_apply`, `Polynomial.coeff_monomial`, etc.
---
- [ ] depends on: #30909
- [ ] depends on: #30911
[](https://gitpod.io/from-referrer/)
|
merge-conflict |
34/81 |
Mathlib/Algebra/Group/Pi/Lemmas.lean,Mathlib/Algebra/Notation/Pi/Basic.lean,Mathlib/Data/Set/Prod.lean,Mathlib/Logic/Embedding/Basic.lean,Mathlib/Logic/Equiv/Basic.lean,Mathlib/Logic/Function/Basic.lean |
6 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
27-74159 27 days ago |
27-74160 27 days ago |
0-0 0 seconds |
| 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
|
421/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 |
25-56424 25 days ago |
104-41890 3 months ago |
17-16247 17 days |
| 25481 |
kbuzzard author:kbuzzard |
chore: refactor Algebra.TensorProduct.rightAlgebra |
The declaration `Algebra.TensorProduct.rightAlgebra` makes `A ⊗[R] B` into a `B`-algebra (here `R` is a `CommSemiring`, `A` is a `Semiring` and an `R`-algebra, and `B` is a `CommSemiring` and an `R`-algebra). It is not an instance because if A = B it causes a diamond. However in the many cases where A isn't B, it can occasionally be useful.
However one could imagine that in the many cases where an R-module `M` also isn't `B`, it might occasionally be useful to make `M ⊗[R] B` into a `B`-module (and indeed I am finding this in FLT). With the current definition of `Algebra.TensorProduct.rightAlgebra` this is difficult to do without causing diamonds in the case when `M` happens to be an `R`-algebra (by which I mean "I failed to do this in finite time").
One fix for this is just to redefine `Algebra.TensorProduct.rightAlgebra` so that the `smul` field is
```
smul b ab := TensorProduct.comm _ _ _ (b • (TensorProduct.comm _ _ _ ab))
```
i.e. literally "swap the product around, use mathlib's instance making `B ⊗[R] A` into a `B`-algebra, and then swap back". Then the same definition can be used to make `M ⊗[R] B` into a `B`-module and on the odd occasion where this point of view is useful, there is no diamond. This is what we do in this PR. After adding one simp lemma there is no breakage at all in mathlib. Furthermore, for those who have observed that we want to build on this algebra instance sometimes and, for example, add instances of the form "if M is finite over R then M ⊗[R] B is finite over B" -- these instances are really easy to add now with this new definition, because you simply pull back the analogous finite left module instance along the isomorphism M ⊗[R] B = B ⊗[R] M. Examples (from FLT, where the right action is put in a scope):
```
scoped instance [Module.Finite R M] : Module.Finite A (M ⊗[R] A) :=
Module.Finite.equiv (Module.TensorProduct.comm R A M)
scoped instance [Module.Free R M] : Module.Free A (M ⊗[R] A) :=
Module.Free.of_equiv (Module.TensorProduct.comm R A M)
```
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
delegated
label:t-algebra$ |
33/6 |
Mathlib/RingTheory/TensorProduct/Basic.lean |
1 |
8 |
['adomani', 'github-actions', 'kbuzzard', 'leanprover-bot', 'mathlib-bors', 'mathlib4-merge-conflict-bot'] |
adomani assignee:adomani |
24-71992 24 days ago |
24-71993 24 days ago |
56-85445 56 days |
| 26827 |
pechersky author:pechersky |
feat(Analysis/Normed/ValuativeRel): helper instance for NormedField |
---
[](https://gitpod.io/from-referrer/)
- [x] depends on: #26713
- [x] depends on: #26826
|
t-algebra
t-analysis
t-number-theory
merge-conflict
label:t-algebra$ |
211/27 |
Mathlib.lean,Mathlib/Analysis/Normed/ValuativeRel.lean,Mathlib/Topology/Algebra/Valued/ValuativeRel.lean |
3 |
34 |
['ADedecker', 'adamtopaz', 'erdOne', 'github-actions', 'kbuzzard', 'kckennylau', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'pechersky'] |
kbuzzard assignee:kbuzzard |
22-65797 22 days ago |
22-65797 22 days ago |
127-58875 127 days |
| 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
merge-conflict
|
35/0 |
Mathlib/Data/List/Scan.lean |
1 |
11 |
['ShreckYe', 'github-actions', 'mathlib4-merge-conflict-bot', 'themathqueen', 'vlad902'] |
pechersky assignee:pechersky |
22-22028 22 days ago |
25-19759 25 days ago |
74-62841 74 days |
| 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
merge-conflict
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 |
13 |
['JovanGerb', 'adomani', 'alreadydone', 'bryangingechen', 'github-actions', 'mathlib4-merge-conflict-bot'] |
bryangingechen assignee:bryangingechen |
22-19751 22 days ago |
22-19752 22 days ago |
98-49698 98 days |
| 30150 |
imbrem author:imbrem |
feat(CategoryTheory/Monoidal): to_additive for MonoidalCategory |
Add `AddMonoidalCategory`, the additive version of `MonoidalCategory`.
To get this to work, I needed to _remove_ the `to_additive` attributes in `Discrete.lean`, since existing code relies on the `AddMonoid M → MonoidalCategory M` instance. For now, we simply implement the additive variants by hand instead.
---
As discussed in #28718; I added an `AddMonoidalCategory` struct and tagged `MonoidalCategory` with `to_additive`, along with the lemmas in `Category.lean`.
I think this is the right approach, since under this framework the "correct" additive version of `Discrete.lean` would be mapping an `AddMonoid` to an `AddMonoidalCategory`.
Next steps would be to:
- Make `monoidal_coherence` and `coherence` support `AddMonoidalCategory`
- Add `CocartesianMonoidalCategory` extending `AddMonoidalCategory`
[](https://gitpod.io/from-referrer/)
|
large-import
awaiting-zulip
new-contributor
t-category-theory
t-meta
merge-conflict
|
444/125 |
Mathlib/CategoryTheory/Monoidal/Category.lean,Mathlib/CategoryTheory/Monoidal/Discrete.lean,Mathlib/Tactic/ToAdditive/GuessName.lean |
3 |
22 |
['JovanGerb', 'YaelDillies', 'github-actions', 'imbrem', 'mathlib4-merge-conflict-bot'] |
nobody |
22-18077 22 days ago |
22-18077 22 days ago |
1-18384 1 day |
| 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
merge-conflict
|
471/0 |
Mathlib.lean,Mathlib/Geometry/Diffeology/Basic.lean,docs/references.bib |
3 |
11 |
['JovanGerb', 'github-actions', 'grunweg', 'lecopivo', 'mathlib4-merge-conflict-bot', 'peabrainiac'] |
grunweg assignee:grunweg |
21-78331 21 days ago |
21-78332 21 days ago |
138-31722 138 days |
| 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
merge-conflict
|
320/17 |
Mathlib/Tactic/GCongr/Core.lean,MathlibTest/GConvert.lean |
2 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
21-47222 21 days ago |
21-47223 21 days ago |
0-0 0 seconds |
| 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
merge-conflict
label:t-algebra$ |
66/21 |
Mathlib/LinearAlgebra/Basis/Basic.lean,Mathlib/LinearAlgebra/Basis/Defs.lean,Mathlib/LinearAlgebra/FreeModule/Basic.lean |
3 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
20-78103 20 days ago |
20-78104 20 days ago |
0-0 0 seconds |
| 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
- [ ] depends on: #30380
|
large-import
t-number-theory
merge-conflict
|
1195/18 |
Mathlib.lean,Mathlib/Analysis/Complex/IntegerCompl.lean,Mathlib/Analysis/Complex/UpperHalfPlane/Basic.lean,Mathlib/Data/Int/Interval.lean,Mathlib/NumberTheory/IntervalSums.lean,Mathlib/NumberTheory/ModularForms/EisensteinSeries/E2/Defs.lean,Mathlib/NumberTheory/ModularForms/EisensteinSeries/E2/Summable.lean,Mathlib/NumberTheory/ModularForms/EisensteinSeries/E2/Transform.lean,Mathlib/NumberTheory/ModularForms/EisensteinSeries/QExpansion.lean,Mathlib/NumberTheory/ModularForms/EisensteinSeries/Summable.lean,Mathlib/NumberTheory/ModularForms/Identities.lean,Mathlib/NumberTheory/TsumDivsorsAntidiagonal.lean,Mathlib/Order/Filter/AtTopBot/Finset.lean,Mathlib/Topology/Algebra/InfiniteSum/Defs.lean,Mathlib/Topology/Algebra/InfiniteSum/NatInt.lean,Mathlib/Topology/Algebra/Monoid/Defs.lean |
16 |
7 |
['CBirkbeck', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
20-65015 20 days ago |
56-52577 1 month ago* |
0-0 0 seconds* |
| 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
|
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 |
20-63335 20 days ago |
unknown |
unknown |
| 31388 |
b-mehta author:b-mehta |
feat(Topology/Order): add unordered versions of topological Rolle's theorem |
To support this, we also add lemmas about extending functions from unordered intervals, and take the liberty of using `variable` more in that file, and removing an `erw`.
The motivation here is that this is useful infrastructure for an unordered/central version of Taylor's theorem, as discussed here: [#maths > Taylor's theorem @ 💬](https://leanprover.zulipchat.com/#narrow/channel/116395-maths/topic/Taylor's.20theorem/near/402571017). As such, this PR also originates from the Exponential Ramsey project.
The PR currently makes a couple of different changes, but the overall diff is relatively small, and helps to motivate some of the changes, so I elected to keep it one PR for now, unless other maintainers would prefer it to be split up or further explained.
|
tech debt
t-analysis
merge-conflict
awaiting-author
|
107/24 |
Mathlib/Order/Interval/Set/UnorderedInterval.lean,Mathlib/Topology/Order/DenselyOrdered.lean,Mathlib/Topology/Order/ExtendFrom.lean,Mathlib/Topology/Order/LeftRight.lean,Mathlib/Topology/Order/Rolle.lean |
5 |
n/a |
['ADedecker', 'b-mehta', 'github-actions', 'j-loreaux', 'mathlib4-merge-conflict-bot', 'mcdoll', 'plp127'] |
nobody |
20-63090 20 days ago |
unknown |
unknown |
| 30978 |
dagurtomas author:dagurtomas |
Draft: adic spaces |
---
This is work in progress, mostly ported from the perfectoid project
[](https://gitpod.io/from-referrer/)
|
large-import
merge-conflict
|
1407/45 |
Mathlib.lean,Mathlib/AdicSpace/AdicSpace.lean,Mathlib/AdicSpace/HuberPair.lean,Mathlib/AdicSpace/Spa/RationalOpenData.lean,Mathlib/AdicSpace/Spa/StalkValuation.lean,Mathlib/AdicSpace/Spa/StructurePresheaf.lean,Mathlib/AdicSpace/Spv.lean,Mathlib/Topology/Category/TopCommRingCat.lean |
8 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
20-58776 20 days ago |
20-58777 20 days ago |
0-0 0 seconds |
| 30706 |
astrainfinita author:astrainfinita |
refactor(Analysis/NormedSpace/Exponential): remove the `𝕂` argument from `exp` |
This PR builds upon #8370 and avoids `Algebra ℚ` typeclass assumptions wherever possible.
Many `[NormedAlgebra ℚ 𝔸]` can be generalized to `[NontriviallyNormedField 𝕂] [CharZero 𝕂] [ContinuousSMul ℚ 𝕂] [NormedAlgebra 𝕂 𝔸]`, which basically means allowing `ℚ` to use other equivalent norms, and may not be the case of concern.
It might be possible to use some Prop-valued typeclasses to avoid the diamond problem potentially caused by `[NormedAlgebra ℚ 𝔸]`. This makes it unnecessary to manually obtain `[NormedAlgebra ℚ 𝔸]` when we have `[NormedAlgebra ℝ 𝔸]` or `[NormedAlgebra ℂ 𝔸]`.
Co-authored-by: Eric Wieser
---
- [ ] depends on: #28475
There are still some documentation comments that need to be updated.
Zulip: [#mathlib4 > Real.exp @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Real.2Eexp/near/401602245)
[](https://gitpod.io/from-referrer/)
|
t-analysis
merge-conflict
awaiting-author
|
477/444 |
Counterexamples/DiscreteTopologyNonDiscreteUniformity.lean,Mathlib/Analysis/CStarAlgebra/Exponential.lean,Mathlib/Analysis/CStarAlgebra/Spectrum.lean,Mathlib/Analysis/CStarAlgebra/Unitary/Connected.lean,Mathlib/Analysis/Normed/Algebra/DualNumber.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/Real/Hyperreal.lean,Mathlib/Analysis/SpecialFunctions/Complex/LogBounds.lean,Mathlib/Analysis/SpecialFunctions/ContinuousFunctionalCalculus/ExpLog.lean,Mathlib/Analysis/SpecialFunctions/Exponential.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Series.lean,Mathlib/Analysis/SpecificLimits/Basic.lean,Mathlib/Analysis/SpecificLimits/RCLike.lean,Mathlib/Combinatorics/Derangements/Exponential.lean,Mathlib/MeasureTheory/Measure/CharacteristicFunction.lean,Mathlib/Probability/Distributions/Gaussian/Basic.lean,Mathlib/Probability/Distributions/Gaussian/Fernique.lean,Mathlib/Probability/Distributions/Poisson.lean |
22 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
20-9129 20 days ago |
36-22591 1 month ago |
0-996 16 minutes |
| 30824 |
grunweg author:grunweg |
wip: another smoothness lemma for local frames |
---
Can I prove in general that the coefficients of a smooth section w.r.t. a smooth local frame are smooth?
This is certainly true for orthonormal frames...
[](https://gitpod.io/from-referrer/)
|
t-differential-geometry
merge-conflict
WIP
|
57/9 |
Mathlib/Geometry/Manifold/VectorBundle/LocalFrame.lean |
1 |
3 |
['github-actions', 'grunweg', 'mathlib4-merge-conflict-bot'] |
nobody |
19-47114 19 days ago |
19-47115 19 days ago |
0-6 6 seconds |
| 30962 |
WangYiran01 author:WangYiran01 |
feat(Combinatorics/Enumerative): add lattice path lemmas and counts |
This PR adds definitions and theorems about monotone lattice paths:
- Defines `pathCount`, `pathCountFrom`, `SubdiagProp`, and related structures.
- Proves closed forms such as `pathCount_eq_closed`.
- Adds Dyck/ballot subdiagonal property (`SubdiagProp`).
All code builds successfully with `lake build`. |
new-contributor
t-combinatorics
merge-conflict
|
64/0 |
Mathlib.lean,Mathlib/Combinatorics/Enumerative/RecLatticePath.lean |
2 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
awainverse assignee:awainverse |
19-33588 19 days ago |
19-33588 19 days ago |
19-55009 19 days |
| 30322 |
kckennylau author:kckennylau |
feat(RingTheory): base change of graded algebra |
In this file we show that if `𝒜` is a graded `R`-algebra, and `S` is any `R`-algebra, then `S ⊗[R] 𝒜` (which is actually `fun i ↦ (𝒜 i).baseChange S`) is a graded `S`-algebra with the same grading.
---
Split from #26061.
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
merge-conflict
awaiting-author
|
272/47 |
Mathlib.lean,Mathlib/Algebra/DirectSum/Basic.lean,Mathlib/Algebra/DirectSum/Decomposition.lean,Mathlib/Algebra/DirectSum/Module.lean,Mathlib/Algebra/Order/Module/HahnEmbedding.lean,Mathlib/LinearAlgebra/DirectSum/Finsupp.lean,Mathlib/LinearAlgebra/DirectSum/TensorProduct.lean,Mathlib/LinearAlgebra/TensorProduct/Decomposition.lean,Mathlib/LinearAlgebra/TensorProduct/Tower.lean,Mathlib/RingTheory/Flat/Basic.lean,Mathlib/RingTheory/Flat/FaithfullyFlat/Basic.lean,Mathlib/RingTheory/GradedAlgebra/TensorProduct.lean |
12 |
11 |
['erdOne', 'github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
18-53372 18 days ago |
18-53373 18 days ago |
36-68500 36 days |
| 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
label:t-algebra$ |
1141/54 |
Mathlib.lean,Mathlib/Algebra/MonoidAlgebra/Basic.lean,Mathlib/Algebra/NoZeroSMulDivisors/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/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 |
18-38064 18 days ago |
unknown |
unknown |
| 30770 |
robertmaxton42 author:robertmaxton42 |
(WIP) Limits and Colimits in Quiv |
WIP PR for the oleans
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict
WIP
|
3652/31 |
Mathlib.lean,Mathlib/CategoryTheory/Category/Quiv.lean,Mathlib/CategoryTheory/Category/Quiv/AsFunctor/Defs.lean,Mathlib/CategoryTheory/Category/Quiv/Colimits.lean,Mathlib/CategoryTheory/Category/Quiv/Limits.lean,Mathlib/CategoryTheory/Category/Quiv/Shapes.lean,Mathlib/CategoryTheory/Category/Quiv/WalkingQuiver.lean,Mathlib/CategoryTheory/EqToHom.lean,Mathlib/CategoryTheory/Equivalence.lean,Mathlib/CategoryTheory/Filtered/Level.lean,Mathlib/CategoryTheory/Limits/Constructions/LimitsOfProductsAndEqualizers.lean,Mathlib/CategoryTheory/Limits/FunctorCategory/Basic.lean,Mathlib/CategoryTheory/Limits/Shapes/FunctorToTypes.lean,Mathlib/CategoryTheory/Limits/Types/Colimits.lean,Mathlib/CategoryTheory/ObjectProperty/FullSubcategory.lean,Mathlib/CategoryTheory/Topos/Classifier.lean,Mathlib/CategoryTheory/Topos/Presheaf.lean,Mathlib/Combinatorics/Quiver/Shapes.lean,Mathlib/Combinatorics/Quiver/WalkingQuiver.lean,Mathlib/Data/ULift.lean,Mathlib/Logic/Equiv/Basic.lean,Mathlib/Logic/Equiv/Sum.lean,Mathlib/Logic/Small/Defs.lean |
23 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
18-17542 18 days ago |
34-77283 1 month ago |
0-0 0 seconds |
| 31593 |
Ruben-VandeVelde author:Ruben-VandeVelde |
feat: some lemmas about MonoidAlgebra |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
awaiting-author
label:t-algebra$ |
26/0 |
Mathlib/Algebra/MonoidAlgebra/Basic.lean |
1 |
5 |
['github-actions', 'mathlib4-merge-conflict-bot', 'robin-carlier', 'themathqueen'] |
nobody |
18-11192 18 days ago |
18-11193 18 days ago |
0-85235 23 hours |
| 31596 |
grunweg author:grunweg |
chore: remove extraneous uses of push_neg |
---
Ideally, repeat this experiment after the new `contrapose!` for equivalences has been merged...
[](https://gitpod.io/from-referrer/)
|
merge-conflict
WIP
|
155/99 |
Mathlib/Algebra/Group/Fin/Basic.lean,Mathlib/Algebra/Group/Pointwise/Finset/Basic.lean,Mathlib/Algebra/Group/Pointwise/Set/Basic.lean,Mathlib/Algebra/Group/UniqueProds/Basic.lean,Mathlib/Algebra/Homology/Embedding/Basic.lean,Mathlib/Algebra/Order/Archimedean/Class.lean,Mathlib/AlgebraicTopology/SimplicialSet/Degenerate.lean,Mathlib/Analysis/SpecialFunctions/BinaryEntropy.lean,Mathlib/CategoryTheory/Limits/Shapes/Preorder/WellOrderContinuous.lean,Mathlib/Combinatorics/Colex.lean,Mathlib/Combinatorics/SimpleGraph/Clique.lean,Mathlib/Combinatorics/SimpleGraph/Metric.lean,Mathlib/Data/EReal/Operations.lean,Mathlib/Data/Nat/Count.lean,Mathlib/Data/Seq/Basic.lean,Mathlib/GroupTheory/Perm/ClosureSwap.lean,Mathlib/GroupTheory/Perm/Cycle/Basic.lean,Mathlib/LinearAlgebra/LinearIndependent/Defs.lean,Mathlib/LinearAlgebra/RootSystem/GeckConstruction/Semisimple.lean,Mathlib/ModelTheory/Semantics.lean,Mathlib/NumberTheory/Padics/PadicVal/Basic.lean,Mathlib/NumberTheory/WellApproximable.lean,Mathlib/Order/LiminfLimsup.lean,Mathlib/RingTheory/HahnSeries/Basic.lean,Mathlib/RingTheory/HahnSeries/Multiplication.lean,Mathlib/RingTheory/Ideal/AssociatedPrime/Basic.lean,Mathlib/RingTheory/Ideal/Oka.lean,Mathlib/RingTheory/Localization/AtPrime/Basic.lean,Mathlib/RingTheory/Valuation/ValuativeRel/Basic.lean,Mathlib/SetTheory/Ordinal/Principal.lean,Mathlib/Tactic/ByCases.lean,Mathlib/Tactic/ByContra.lean,Mathlib/Tactic/Contrapose.lean,Mathlib/Tactic/NormNum/Core.lean,Mathlib/Tactic/Push.lean,Mathlib/Topology/LocallyFinsupp.lean,Mathlib/Topology/Maps/Basic.lean,Mathlib/Topology/Separation/Regular.lean,Mathlib/Util/AtLocation.lean,MathlibTest/Contrapose.lean,MathlibTest/byContra.lean,MathlibTest/push_neg.lean |
42 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
18-3482 18 days ago |
18-3483 18 days ago |
0-1 1 second |
| 31600 |
grunweg author:grunweg |
chore: replace by_cases! with by_cases when the push_neg step does no… |
…thing
Not exhaustive yet.
---
Spun out of #31596.
[](https://gitpod.io/from-referrer/)
|
merge-conflict
WIP
|
29/29 |
Mathlib/Algebra/Group/Fin/Basic.lean,Mathlib/Algebra/Homology/Embedding/Basic.lean,Mathlib/Algebra/Order/Archimedean/Class.lean,Mathlib/AlgebraicTopology/SimplicialSet/Degenerate.lean,Mathlib/CategoryTheory/Limits/Shapes/Preorder/WellOrderContinuous.lean,Mathlib/Combinatorics/Colex.lean,Mathlib/Combinatorics/SimpleGraph/Clique.lean,Mathlib/Combinatorics/SimpleGraph/Metric.lean,Mathlib/Data/Seq/Basic.lean,Mathlib/GroupTheory/Perm/ClosureSwap.lean,Mathlib/GroupTheory/Perm/Cycle/Basic.lean,Mathlib/ModelTheory/Semantics.lean,Mathlib/Order/LiminfLimsup.lean,Mathlib/RingTheory/HahnSeries/Basic.lean,Mathlib/RingTheory/HahnSeries/Multiplication.lean,Mathlib/RingTheory/Ideal/AssociatedPrime/Basic.lean,Mathlib/RingTheory/Ideal/Oka.lean,Mathlib/RingTheory/Localization/AtPrime/Basic.lean,Mathlib/RingTheory/Valuation/ValuativeRel/Basic.lean,Mathlib/SetTheory/Ordinal/Principal.lean,Mathlib/Topology/Maps/Basic.lean |
21 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
18-3481 18 days ago |
18-3482 18 days ago |
0-2 2 seconds |
| 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
merge-conflict
|
229/0 |
Mathlib.lean,Mathlib/Geometry/Manifold/SliceModel.lean |
2 |
4 |
['github-actions', 'grunweg', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
17-37196 17 days ago |
17-37197 17 days ago |
146-23442 146 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
merge-conflict
|
14/15 |
Mathlib/Tactic/Linter/CommandStart.lean |
1 |
6 |
['github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'mathlib4-merge-conflict-bot'] |
joneugster assignee:joneugster |
16-73074 16 days ago |
16-73075 16 days ago |
150-52942 150 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/)
|
file-removed
large-import
t-meta
merge-conflict
awaiting-author
|
210277/112616 |
.github/PULL_REQUEST_TEMPLATE.md,.github/actionlint.yml,.github/build.in.yml,.github/workflows/PR_summary.yml,.github/workflows/actionlint.yml,.github/workflows/add_label_from_diff.yaml,.github/workflows/auto_assign_reviewers.yaml,.github/workflows/bench_summary_comment.yml,.github/workflows/bors.yml,.github/workflows/bot_fix_style.yaml,.github/workflows/build.yml,.github/workflows/build_fork.yml,.github/workflows/daily.yml,.github/workflows/discover-lean-pr-testing.yml,.github/workflows/docker_build.yml,.github/workflows/label_new_contributor.yml,.github/workflows/latest_import.yml,.github/workflows/lint_and_suggest_pr.yml,.github/workflows/long_file_report.yml,.github/workflows/maintainer_bors.yml,.github/workflows/maintainer_bors_wf_run.yml,.github/workflows/maintainer_merge.yml,.github/workflows/maintainer_merge_wf_run.yml,.github/workflows/mk_build_yml.sh,.github/workflows/nightly-docgen.yml,.github/workflows/nightly-regression-report.yml,.github/workflows/nightly_bump_toolchain.yml,.github/workflows/nightly_detect_failure.yml,.github/workflows/nightly_merge_master.yml,.github/workflows/nolints.yml,.github/workflows/pre-commit.yml,.github/workflows/remove_deprecated_decls.yml,.github/workflows/stale.yml,.github/workflows/technical_debt_metrics.yml,.github/workflows/update_dependencies.yml,.github/workflows/update_dependencies_zulip.yml,.github/workflows/weekly-lints.yml,.github/workflows/zulip_emoji_closed_pr.yaml,.github/workflows/zulip_emoji_labelling.yaml,.github/workflows/zulip_emoji_merge_delegate.yaml,.pre-commit-config.yaml,Archive.lean,Archive/Arithcc.lean,Archive/Examples/Eisenstein.lean,Archive/Examples/IfNormalization/Result.lean,Archive/Examples/IfNormalization/Statement.lean,Archive/Examples/IfNormalization/WithoutAesop.lean,Archive/Examples/Kuratowski.lean,Archive/Examples/MersennePrimes.lean,Archive/Imo/Imo1959Q2.lean,Archive/Imo/Imo1960Q1.lean,Archive/Imo/Imo1961Q3.lean,Archive/Imo/Imo1962Q1.lean,Archive/Imo/Imo1962Q4.lean,Archive/Imo/Imo1972Q5.lean,Archive/Imo/Imo1975Q1.lean,Archive/Imo/Imo1981Q3.lean,Archive/Imo/Imo1982Q1.lean,Archive/Imo/Imo1982Q3.lean,Archive/Imo/Imo1987Q1.lean,Archive/Imo/Imo1994Q1.lean,Archive/Imo/Imo1997Q3.lean,Archive/Imo/Imo1998Q2.lean,Archive/Imo/Imo2001Q2.lean,Archive/Imo/Imo2001Q3.lean,Archive/Imo/Imo2001Q4.lean,Archive/Imo/Imo2001Q5.lean,Archive/Imo/Imo2005Q3.lean,Archive/Imo/Imo2005Q4.lean,Archive/Imo/Imo2006Q3.lean,Archive/Imo/Imo2008Q2.lean,Archive/Imo/Imo2008Q4.lean,Archive/Imo/Imo2011Q3.lean,Archive/Imo/Imo2013Q1.lean,Archive/Imo/Imo2013Q5.lean,Archive/Imo/Imo2015Q6.lean,Archive/Imo/Imo2019Q2.lean,Archive/Imo/Imo2021Q1.lean,Archive/Imo/Imo2024Q1.lean,Archive/Imo/Imo2024Q3.lean,Archive/Imo/Imo2024Q5.lean,Archive/Imo/Imo2024Q6.lean,Archive/Imo/README.md,Archive/Kuratowski.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/HeronsFormula.lean,Archive/Wiedijk100Theorems/InverseTriangleSum.lean,Archive/Wiedijk100Theorems/Partition.lean,Archive/Wiedijk100Theorems/PerfectNumbers.lean,Archive/Wiedijk100Theorems/SolutionOfCubicQuartic.lean,Archive/Wiedijk100Theorems/SumOfPrimeReciprocalsDiverges.lean,Cache/IO.lean,Cache/Main.lean |
5782 |
14 |
['Paul-Lez', 'Vierkantor', 'eric-wieser', 'github-actions', 'kmill', 'mathlib4-merge-conflict-bot'] |
nobody |
16-52022 16 days ago |
55-72952 1 month ago* |
67-54211 67 days* |
| 29909 |
Vierkantor author:Vierkantor |
feat(CI): add build output to CI workflows |
This PR uses the Zulip build report script (originally developed for the nightly-regression-report workflow) to add a summary of build output to other Zulip posts about workflow results. This allows us to more easily see the origin of a failure. This requires redoing the script a little to make it a bit more flexible, and the output is slightly reformatted to become consistent across the various workflows (4 of them that post to Zulip).
We don't do so for the nightly-testing failures, since those run in a different workflow, and it would be a lot of work to access the command output from another workflow.
---
[](https://gitpod.io/from-referrer/)
|
CI
merge-conflict
|
93/69 |
.github/workflows/daily.yml,.github/workflows/nightly-docgen.yml,.github/workflows/nightly-regression-report.yml,scripts/zulip_build_report.sh |
4 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
16-52021 16 days ago |
31-15503 1 month ago |
41-48286 41 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/)
|
merge-conflict |
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 |
7 |
['github-actions', 'grunweg', 'kbuzzard', 'mathlib4-merge-conflict-bot'] |
nobody |
16-50822 16 days ago |
21-61584 21 days ago |
98-27129 98 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
merge-conflict
awaiting-author
|
37/0 |
Mathlib/Data/Matrix/Invertible.lean |
1 |
5 |
['eric-wieser', 'github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
16-2219 16 days ago |
16-2220 16 days ago |
23-30991 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
merge-conflict
|
490/0 |
Mathlib.lean,Mathlib/Computability/RegularExpressionsToEpsilonNFA.lean,docs/references.bib |
3 |
7 |
['anthonyde', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'meithecatte', 'qawbecrdtey'] |
nobody |
16-2218 16 days ago |
16-2219 16 days ago |
75-77754 75 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
merge-conflict
WIP
|
175/0 |
Mathlib/ModelTheory/Graph.lean,Mathlib/ModelTheory/Substructures.lean |
2 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
16-2216 16 days ago |
16-2217 16 days 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
merge-conflict
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 |
42 |
['alreadydone', 'github-actions', 'jcommelin', 'jjaassoonn', 'kbuzzard', 'mathlib4-merge-conflict-bot', 'qawbecrdtey'] |
nobody |
16-2215 16 days ago |
16-2216 16 days ago |
20-7596 20 days |
| 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
merge-conflict
|
305/0 |
Mathlib.lean,Mathlib/Computability/QueryComplexity/Basic.lean,Mathlib/Computability/QueryComplexity/Defs.lean |
3 |
60 |
['eric-wieser', 'girving', 'github-actions', 'mathlib4-merge-conflict-bot', 'quangvdao', 'tomaz1502'] |
nobody |
16-2214 16 days ago |
16-2214 16 days ago |
300-54997 300 days |
| 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
merge-conflict
awaiting-author
|
102/0 |
Mathlib/ModelTheory/Bundled.lean |
1 |
27 |
['GabinKolly', 'Vierkantor', 'YaelDillies', 'github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
16-2210 16 days ago |
16-2211 16 days ago |
50-58472 50 days |
| 21447 |
erdOne author:erdOne |
feat(AlgebraicGeometry): the split algebraic torus |
---
[](https://gitpod.io/from-referrer/)
|
t-algebraic-geometry
merge-conflict
awaiting-author
|
419/0 |
Mathlib.lean,Mathlib/AlgebraicGeometry/Torus.lean |
2 |
5 |
['erdOne', 'github-actions', 'joelriou', 'mathlib4-merge-conflict-bot'] |
nobody |
16-2207 16 days ago |
16-2208 16 days ago |
2-69252 2 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
merge-conflict
awaiting-author
|
229/0 |
Mathlib.lean,Mathlib/Topology/Path/CountableConcat.lean |
2 |
31 |
['YaelDillies', 'github-actions', 'kim-em', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'peabrainiac'] |
YaelDillies assignee:YaelDillies |
16-2205 16 days ago |
16-2206 16 days ago |
56-56728 56 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
merge-conflict
awaiting-author
|
144/0 |
Mathlib.lean,Mathlib/CategoryTheory/Pi/Basic.lean,Mathlib/CategoryTheory/Pi/Monoidal.lean,Mathlib/CategoryTheory/Pi/MonoidalClosed.lean |
4 |
20 |
['TwoFX', 'YaelDillies', 'b-mehta', 'github-actions', 'jcommelin', 'mathlib4-merge-conflict-bot', 'sinhp'] |
nobody |
16-2204 16 days ago |
16-2205 16 days ago |
54-54882 54 days |
| 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
merge-conflict
awaiting-author
label:t-algebra$ |
174/0 |
Mathlib.lean,Mathlib/LinearAlgebra/TensorProduct/HomTensor.lean |
2 |
27 |
['Whysoserioushah', 'YaelDillies', 'erdOne', 'github-actions', 'kbuzzard', 'mathlib4-merge-conflict-bot'] |
nobody |
16-2202 16 days ago |
16-2203 16 days ago |
46-53384 46 days |
| 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
merge-conflict
label:t-algebra$ |
169/0 |
Mathlib/Algebra/Free.lean |
1 |
12 |
['YaelDillies', 'github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
16-2078 16 days ago |
16-2079 16 days ago |
51-9403 51 days |
| 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
merge-conflict
awaiting-author
|
70/0 |
Mathlib.lean,Mathlib/Computability/PDA.lean |
2 |
35 |
['YaelDillies', 'github-actions', 'madvorak', 'mathlib4-merge-conflict-bot', 'shetzl'] |
nobody |
16-2072 16 days ago |
16-2073 16 days ago |
20-81771 20 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
merge-conflict
|
698/0 |
Archive/Examples/SumOracle.lean,Mathlib.lean,Mathlib/Computability/QueryComplexity/Defs.lean,Mathlib/Computability/QueryComplexity/Sort.lean |
4 |
5 |
['eric-wieser', 'girving', 'github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
16-2069 16 days ago |
16-2071 16 days ago |
0-0 0 seconds |
| 22231 |
pechersky author:pechersky |
feat(Algebra/Valued): `AdicExpansion` initial defns |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-topology
merge-conflict
awaiting-author
label:t-algebra$ |
299/0 |
Mathlib.lean,Mathlib/Topology/Algebra/Valued/AdicExpansion.lean |
2 |
8 |
['Thmoas-Guan', 'github-actions', 'grunweg', 'jcommelin', 'mathlib4-merge-conflict-bot'] |
jcommelin assignee:jcommelin |
16-2068 16 days ago |
16-2069 16 days ago |
189-33553 189 days |
| 22302 |
658060 author:658060 |
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
merge-conflict
awaiting-author
|
312/0 |
Mathlib.lean,Mathlib/CategoryTheory/Topos/Power.lean |
2 |
3 |
['github-actions', 'joelriou', 'mathlib4-merge-conflict-bot'] |
b-mehta assignee:b-mehta |
16-2063 16 days ago |
16-2064 16 days ago |
0-1528 25 minutes |
| 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
merge-conflict
awaiting-author
|
383/0 |
Mathlib.lean,Mathlib/Computability/LeftmostDerivation.lean |
2 |
55 |
['YaelDillies', 'github-actions', 'madvorak', 'mathlib4-merge-conflict-bot', 'shetzl'] |
YaelDillies assignee:YaelDillies |
16-2061 16 days ago |
16-2062 16 days ago |
72-3718 72 days |
| 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
merge-conflict
WIP
|
167/0 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter.lean,Mathlib/Tactic/Linter/VariableVariable.lean,variableDeclarationVariable_replacements.py |
5 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
16-2059 16 days ago |
16-2060 16 days 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
merge-conflict
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 |
8 |
['github-actions', 'mathlib4-merge-conflict-bot', 'mergify'] |
nobody |
16-2057 16 days ago |
16-2059 16 days ago |
0-0 0 seconds |
| 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
merge-conflict
label:t-algebra$ |
74/0 |
Mathlib/RingTheory/Localization/Away/Basic.lean |
1 |
18 |
['eric-wieser', 'github-actions', 'grunweg', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'plp127', 'vihdzp'] |
kim-em assignee:kim-em |
16-2056 16 days ago |
16-2057 16 days ago |
257-28368 257 days |
| 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
merge-conflict
awaiting-author
|
111/1 |
Mathlib/Analysis/Calculus/Deriv/Basic.lean,Mathlib/Analysis/Calculus/IteratedDeriv/Lemmas.lean,Mathlib/Analysis/Calculus/Taylor.lean |
3 |
13 |
['Paul-Lez', 'github-actions', 'grunweg', 'mathlib4-merge-conflict-bot', 'mhk119'] |
nobody |
16-2050 16 days ago |
16-2051 16 days ago |
30-77130 30 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
merge-conflict
awaiting-author
label:t-algebra$ |
100/0 |
Mathlib.lean,Mathlib/LinearAlgebra/BilinearForm/Trace.lean |
2 |
4 |
['github-actions', 'jcommelin', 'mathlib4-merge-conflict-bot'] |
nobody |
16-2048 16 days ago |
16-2049 16 days ago |
23-44995 23 days |
| 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
merge-conflict
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 |
31 |
['IvanRenison', 'b-mehta', 'eric-wieser', 'fpvandoorn', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'plp127'] |
b-mehta assignee:b-mehta |
16-2046 16 days ago |
16-2047 16 days ago |
73-73341 73 days |
| 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
merge-conflict
|
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 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-merge-conflict-bot'] |
nobody |
16-2045 16 days ago |
16-2046 16 days ago |
186-81237 186 days |
| 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
merge-conflict
WIP
label:t-algebra$ |
111/45 |
Mathlib/Order/DirectedInverseSystem.lean |
1 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
16-2039 16 days ago |
16-2041 16 days ago |
0-24 24 seconds |
| 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
merge-conflict
WIP
|
205/2 |
Mathlib/Data/ENat/Basic.lean,Mathlib/Data/Set/Card.lean,Mathlib/Topology/Instances/ENat.lean |
3 |
3 |
['eric-wieser', 'github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
16-2035 16 days ago |
16-2037 16 days ago |
14-6036 14 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
merge-conflict
WIP
|
148/0 |
Mathlib.lean,Mathlib/Order/Filter/AtMaxMin.lean |
2 |
5 |
['github-actions', 'mathlib4-merge-conflict-bot', 'plp127', 'urkud'] |
nobody |
16-2034 16 days ago |
16-2035 16 days 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
merge-conflict
awaiting-author
label:t-algebra$ |
138/3 |
Mathlib/LinearAlgebra/Span/Basic.lean,Mathlib/Topology/Algebra/LinearTopology.lean |
2 |
22 |
['ADedecker', 'AntoineChambert-Loir', 'erdOne', 'github-actions', 'grunweg', 'mathlib4-merge-conflict-bot'] |
ADedecker and AntoineChambert-Loir assignee:AntoineChambert-Loir assignee:ADedecker |
16-2032 16 days ago |
16-2033 16 days ago |
124-78308 124 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
merge-conflict
awaiting-author
|
241/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 |
11 |
['chrisflav', 'erdOne', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
grunweg assignee:grunweg |
16-2030 16 days ago |
16-2031 16 days ago |
67-2437 67 days |
| 24129 |
urkud author:urkud |
feat: symmetry of Gateaux derivatives |
---
[](https://gitpod.io/from-referrer/)
|
t-analysis
merge-conflict
|
190/1 |
Mathlib.lean,Mathlib/Analysis/Calculus/LineDeriv/Basic.lean,Mathlib/Analysis/Calculus/LineDeriv/Symmetric.lean |
3 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
16-1900 16 days ago |
16-1901 16 days ago |
0-0 0 seconds |
| 24161 |
urkud author:urkud |
feat(Analysis/Calculus/Schwarzian): new file |
---
[](https://gitpod.io/from-referrer/)
|
t-analysis
merge-conflict
|
190/3 |
Mathlib.lean,Mathlib/Analysis/Calculus/Deriv/ZPow.lean,Mathlib/Analysis/Calculus/Schwarzian/Basic.lean |
3 |
3 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-merge-conflict-bot'] |
nobody |
16-1898 16 days ago |
16-1900 16 days ago |
0-0 0 seconds |
| 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
merge-conflict
awaiting-author
|
187/0 |
Mathlib.lean,Mathlib/Combinatorics/SimpleGraph/Cycle.lean |
2 |
42 |
['IvanRenison', 'github-actions', 'mathlib4-merge-conflict-bot', 'vlad902'] |
kmill assignee:kmill |
16-1897 16 days ago |
16-1898 16 days ago |
123-22718 123 days |
| 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
merge-conflict
awaiting-author
|
129/1 |
Mathlib.lean,Mathlib/Data/List/Commutativity.lean,Mathlib/Data/List/Defs.lean,Mathlib/Data/List/Lemmas.lean |
4 |
36 |
['MrSumato', 'github-actions', 'grunweg', 'mathlib4-merge-conflict-bot', 'plp127'] |
grunweg assignee:grunweg |
16-1894 16 days ago |
16-1895 16 days ago |
29-59355 29 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
merge-conflict
awaiting-author
|
370/0 |
Mathlib.lean,Mathlib/CategoryTheory/Category/Quiv/Shapes.lean,Mathlib/CategoryTheory/Category/Quiv/WalkingQuiver.lean,Mathlib/Logic/Small/Defs.lean |
4 |
14 |
['github-actions', 'joelriou', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'robertmaxton42', 'robin-carlier'] |
nobody |
16-1892 16 days ago |
16-1893 16 days ago |
0-80193 22 hours |
| 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/)
|
merge-conflict
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 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
16-1887 16 days ago |
16-1888 16 days ago |
0-0 0 seconds |
| 24789 |
Ruben-VandeVelde author:Ruben-VandeVelde |
chore: move Algebra.Group.Hom.End to Algebra.Ring |
This moves us towards the goal of not depending on `Ring` under `Algebra.Group`; this is mentioned in https://github.com/leanprover-community/mathlib4/issues/11757 and on [Zulip](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Call.20for.20help.3A.20technical.2F.20organisational.20debt/near/512348574).
---
[](https://gitpod.io/from-referrer/)
|
file-removed
t-algebra
merge-conflict
awaiting-author
label:t-algebra$ |
4/10 |
Mathlib.lean,Mathlib/Algebra/Group/Hom/Instances.lean,Mathlib/Algebra/Module/End.lean,Mathlib/Algebra/MonoidAlgebra/Division.lean,Mathlib/Algebra/Ring/Hom/End.lean |
5 |
10 |
['Ruben-VandeVelde', 'YaelDillies', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-merge-conflict-bot', 'riccardobrasca'] |
riccardobrasca assignee:riccardobrasca |
16-1885 16 days ago |
16-1886 16 days ago |
14-7845 14 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
merge-conflict
|
509/1 |
Mathlib.lean,Mathlib/Topology/MetricSpace/BundledFun.lean,Mathlib/Topology/UniformSpace/Ultra/Pseudometrizable.lean |
3 |
9 |
['ADedecker', 'fpvandoorn', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'pechersky'] |
urkud assignee:urkud |
16-1884 16 days ago |
16-1885 16 days ago |
177-43425 177 days |
| 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
merge-conflict
awaiting-author
label:t-algebra$ |
137/16 |
Mathlib/Data/DFinsupp/Defs.lean,Mathlib/LinearAlgebra/DFinsupp.lean |
2 |
13 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'pechersky'] |
pechersky assignee:pechersky |
16-1879 16 days ago |
16-1880 16 days ago |
19-26510 19 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
merge-conflict
|
141/0 |
Mathlib.lean,Mathlib/Analysis/PDE/Quasilinear/Defs.lean |
2 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
16-1878 16 days ago |
16-1879 16 days ago |
0-0 0 seconds |
| 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
merge-conflict
delegated
awaiting-author
|
75/3 |
Mathlib/Util/Delaborators.lean,Mathlib/Util/PPOptions.lean,MathlibTest/delaborators.lean |
3 |
19 |
['JovanGerb', 'Rob23oba', 'eric-wieser', 'github-actions', 'kmill', 'mathlib-bors', 'mathlib4-merge-conflict-bot', 'plp127'] |
alexjbest assignee:alexjbest |
16-1754 16 days ago |
16-1755 16 days ago |
83-71907 83 days |
| 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
merge-conflict
awaiting-author
|
105/0 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter/DeprecatedSimpLemma.lean,MathlibTest/DeprecatedSimpLemmaTest.lean |
4 |
8 |
['adomani', 'github-actions', 'grunweg', 'mathlib4-merge-conflict-bot'] |
nobody |
16-1752 16 days ago |
16-1753 16 days ago |
0-34675 9 hours |
| 25683 |
eric-wieser author:eric-wieser |
feat: Enumeration of NonemptyInterval |
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-data
merge-conflict
|
52/4 |
Mathlib/Data/Sym/Sym2/Fin.lean,Mathlib/Data/Sym/Sym2/Order.lean |
2 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
16-1749 16 days ago |
16-1750 16 days ago |
0-0 0 seconds |
| 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
merge-conflict
awaiting-author
|
217/0 |
Mathlib.lean,Mathlib/NumberTheory/LegendreSymbol/Basic.lean,Mathlib/NumberTheory/LegendreSymbol/QuadraticReciprocity.lean,Mathlib/NumberTheory/LegendreSymbol/QuadraticResidueRoots.lean |
4 |
3 |
['github-actions', 'kckennylau', 'mathlib4-merge-conflict-bot'] |
literandltx assignee:literandltx |
16-1748 16 days ago |
16-1749 16 days ago |
17-63153 17 days |
| 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
merge-conflict
awaiting-author
|
162/0 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/CategoryTheory/RotateIsos/Cancelable.lean,scripts/noshake.json |
4 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
16-1746 16 days ago |
16-1747 16 days ago |
0-0 0 seconds |
| 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
merge-conflict
awaiting-author
|
178/0 |
Mathlib.lean,Mathlib/CategoryTheory/Bicategory/LocallyGroupoid.lean,Mathlib/CategoryTheory/Core.lean |
3 |
9 |
['b-mehta', 'github-actions', 'joelriou', 'mathlib4-merge-conflict-bot', 'robin-carlier'] |
joelriou assignee:joelriou |
16-1737 16 days ago |
16-1738 16 days ago |
105-83970 105 days |
| 25838 |
Bergschaf author:Bergschaf |
feat(Order/Atoms): Finsets are Atomistic |
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-order
merge-conflict
|
31/0 |
Mathlib/Order/Atoms.lean |
1 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
16-1727 16 days ago |
16-1728 16 days ago |
0-0 0 seconds |
| 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
merge-conflict
awaiting-author
|
77/8 |
Mathlib/Algebra/Polynomial/Coeff.lean,Mathlib/RingTheory/Polynomial/SmallDegreeVieta.lean |
2 |
47 |
['chrisflav', 'github-actions', 'kckennylau', 'mans0954', 'mathlib4-merge-conflict-bot', 'ocfnash'] |
chrisflav assignee:chrisflav |
16-1722 16 days ago |
16-1723 16 days ago |
82-34290 82 days |
| 25974 |
scholzhannah author:scholzhannah |
feat(Topology/Compactness/CompactlyCoherentSpace): compact coherentification (k-ification) |
This PR defines the notion of turning an arbitrary topological space into a compactly coherent space. Compactly coherent spaces are commonly referred to as "compactly generated spaces" or "k-spaces" in the literature while the operation of turning a space into such as space is called the "k-ification". There are however three different notions that are described with this name. To disambiguate we use the names "compactly coherent space" and "compactcoherentification" here. See [this wikipedia page](https://en.wikipedia.org/wiki/Compactly_generated_space) for an explanation of these notions.
This PR continues the work from #25318.
Original PR: https://github.com/leanprover-community/mathlib4/pull/25318
Co-authored-by: Floris van Doorn |
large-import
t-topology
merge-conflict
|
174/5 |
Mathlib/Topology/Compactness/CompactlyCoherentSpace.lean |
1 |
5 |
['github-actions', 'joelriou', 'mathlib4-merge-conflict-bot', 'scholzhannah'] |
ADedecker assignee:ADedecker |
16-1716 16 days ago |
16-1717 16 days ago |
148-47112 148 days |
| 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
merge-conflict
|
0/12 |
Mathlib.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Group.lean |
2 |
n/a |
['Multramate', 'github-actions', 'grunweg', 'mathlib4-merge-conflict-bot'] |
nobody |
16-1715 16 days ago |
unknown |
unknown |
| 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
merge-conflict
awaiting-author
|
259/37 |
Mathlib/NumberTheory/EllipticDivisibilitySequence.lean |
1 |
9 |
['MichaelStollBayreuth', 'Multramate', 'github-actions', 'mathlib4-merge-conflict-bot', 'tb65536'] |
tb65536 assignee:tb65536 |
16-1713 16 days ago |
16-1714 16 days ago |
45-1019 45 days |
| 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
merge-conflict
|
265/45 |
Mathlib/NumberTheory/EllipticDivisibilitySequence.lean |
1 |
3 |
['Multramate', 'github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
16-1712 16 days ago |
16-1713 16 days ago |
0-0 0 seconds |
| 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
merge-conflict
WIP
|
289/71 |
Mathlib.lean,Mathlib/GroupTheory/SpecificGroups/Alternating.lean,Mathlib/GroupTheory/SpecificGroups/Alternating/Simple.lean,Mathlib/GroupTheory/Subgroup/Simple.lean |
4 |
14 |
['Komyyy', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'tb65536'] |
nobody |
16-1707 16 days ago |
16-1708 16 days ago |
10-66608 10 days |
| 26158 |
upobir author:upobir |
feat(NumberTheory/Divisors): add int divisors |
This PR continues the work from #25209.
Original PR: https://github.com/leanprover-community/mathlib4/pull/25209 |
t-number-theory
merge-conflict
awaiting-author
|
101/4 |
Mathlib/NumberTheory/Divisors.lean |
1 |
37 |
['MichaelStollBayreuth', 'github-actions', 'mathlib4-merge-conflict-bot', 'upobir'] |
mariainesdff assignee:mariainesdff |
16-1562 16 days ago |
16-1563 16 days ago |
46-1067 46 days |
| 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
merge-conflict
awaiting-author
|
198/2 |
Mathlib/MeasureTheory/Measure/TightNormed.lean |
1 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
16-1540 16 days ago |
16-1540 16 days 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
merge-conflict
WIP
|
352/2 |
Mathlib.lean,Mathlib/MeasureTheory/Measure/TightCharFun.lean,Mathlib/MeasureTheory/Measure/TightNormed.lean |
3 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
16-1538 16 days ago |
16-1539 16 days ago |
0-2 2 seconds |
| 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
merge-conflict
awaiting-author
WIP
|
63/1 |
Mathlib.lean,Mathlib/Data/Array/Extract.lean,Mathlib/New.lean,Mathlib/Tactic/Linter/CommandStart.lean |
4 |
21 |
['adomani', 'bryangingechen', 'github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
16-1537 16 days ago |
16-1538 16 days ago |
0-0 0 seconds |
| 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
merge-conflict
awaiting-author
WIP
|
468/0 |
Mathlib.lean,Mathlib/Analysis/Calculus/FDeriv/Partial.lean,Mathlib/Analysis/Normed/Operator/BoundedLinearMaps.lean |
3 |
21 |
['YaelDillies', 'agjftucker', 'github-actions', 'igorkhavkine', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'sgouezel'] |
sgouezel assignee:sgouezel |
16-1536 16 days ago |
16-1537 16 days ago |
50-22679 50 days |
| 26307 |
j-loreaux author:j-loreaux |
refactor: make `IsIdempotentElem` a one-field structure |
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebra
merge-conflict
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 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
16-1535 16 days ago |
16-1535 16 days ago |
0-0 0 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
merge-conflict
awaiting-author
label:t-algebra$ |
100/0 |
Mathlib.lean,Mathlib/Algebra/Clone/Defs.lean |
2 |
4 |
['Timeroot', 'YaelDillies', 'github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
16-1532 16 days ago |
16-1533 16 days ago |
0-21917 6 hours |
| 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 |
t-logic
merge-conflict
|
145/0 |
Mathlib/Data/Rel.lean,Mathlib/ModelTheory/Definability.lean,scripts/noshake.json |
3 |
30 |
['Timeroot', 'github-actions', 'mathlib4-merge-conflict-bot', 'staroperator'] |
fpvandoorn assignee:fpvandoorn |
16-1531 16 days ago |
16-1532 16 days ago |
145-80722 145 days |
| 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
merge-conflict
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 |
3 |
['github-actions', 'mans0954', 'mathlib4-merge-conflict-bot'] |
nobody |
16-1530 16 days ago |
16-1530 16 days ago |
148-2430 148 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
merge-conflict
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', 'mathlib4-merge-conflict-bot'] |
nobody |
16-1528 16 days ago |
unknown |
unknown |
| 26346 |
mans0954 author:mans0954 |
feat(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
merge-conflict
WIP
label:t-algebra$ |
105/5 |
Mathlib/LinearAlgebra/Basis/Bilinear.lean,Mathlib/LinearAlgebra/QuadraticForm/TensorProduct.lean |
2 |
3 |
['github-actions', 'mans0954', 'mathlib4-merge-conflict-bot'] |
nobody |
16-1527 16 days ago |
16-1528 16 days ago |
0-0 0 seconds |
| 26347 |
mans0954 author:mans0954 |
feat(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
merge-conflict
|
30/0 |
Mathlib.lean,Mathlib/Algebra/Order/Group/Unbundled/Abs.lean,Mathlib/Data/Finset/RangeDistance.lean |
3 |
3 |
['github-actions', 'mans0954', 'mathlib4-merge-conflict-bot'] |
alreadydone assignee:alreadydone |
16-1526 16 days ago |
16-1527 16 days ago |
148-922 148 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
merge-conflict
awaiting-author
|
81/0 |
Mathlib.lean,Mathlib/RingTheory/TwoSidedIdeal/SpanAsSum.lean |
2 |
6 |
['github-actions', 'kckennylau', 'mathlib4-merge-conflict-bot'] |
YaelDillies assignee:YaelDillies |
16-1525 16 days ago |
16-1525 16 days ago |
37-40835 37 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
merge-conflict
please-adopt
|
618/0 |
Mathlib.lean,Mathlib/ModelTheory/FunctionalFormula.lean |
2 |
13 |
['ChrisHughes24', 'github-actions', 'jcommelin', 'kckennylau', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'staroperator'] |
nobody |
16-1519 16 days ago |
16-1520 16 days ago |
125-6199 125 days |
| 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
merge-conflict
|
201/0 |
Mathlib.lean,Mathlib/Data/Nat/LogFueled.lean |
2 |
3 |
['AntoineChambert-Loir', 'github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
16-1517 16 days ago |
16-1518 16 days ago |
145-77007 145 days |
| 26594 |
metakunt author:metakunt |
feat(Algebra/Polynomial/ZMod): Add Polynomial.equiv_of_nat_of_polynomial_zmod |
This adds an explicit bijection between the naturals and $$\mathbb{Z}/n\mathbb{Z}[X]$$ in a canonical way.
---
I feel that some API is missing to make the theorem shorter, I have no idea what lemmas to extract though.
Also I don't know when to use spaces and when not, so I did it best effort.
|
new-contributor
t-algebra
merge-conflict
awaiting-author
label:t-algebra$ |
465/0 |
Mathlib.lean,Mathlib/Algebra/Polynomial/ZMod.lean |
2 |
3 |
['Ruben-VandeVelde', 'github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
16-1388 16 days ago |
16-1389 16 days ago |
25-6199 25 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
merge-conflict
awaiting-author
|
381/0 |
Mathlib.lean,Mathlib/SetTheory/ZFC/Axioms.lean,docs/references.bib |
3 |
50 |
['b-mehta', 'digama0', 'github-actions', 'kckennylau', 'leanprover-community-bot-assistant', 'mathlib4-merge-conflict-bot', 'staroperator', 'vihdzp'] |
b-mehta assignee:b-mehta |
16-1386 16 days ago |
16-1387 16 days ago |
40-53883 40 days |
| 26648 |
eric-wieser author:eric-wieser |
chore(TensorProduct): remove more `suppress_compilation`s |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
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 |
5 |
['eric-wieser', 'github-actions', 'leanprover-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
16-1385 16 days ago |
16-1386 16 days ago |
3-19989 3 days |
| 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
merge-conflict
awaiting-author
|
401/66 |
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 |
17 |
['fweth', 'github-actions', 'joelriou', 'leanprover-community-bot-assistant', 'mathlib4-merge-conflict-bot'] |
joelriou assignee:joelriou |
16-1383 16 days ago |
16-1384 16 days ago |
62-83085 62 days |
| 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
merge-conflict
awaiting-author
|
341/0 |
Mathlib.lean,Mathlib/Analysis/Calculus/PartialDerivativeTest.lean |
2 |
13 |
['bjoernkjoshanssen', 'github-actions', 'j-loreaux', 'mathlib4-merge-conflict-bot', 'themathqueen'] |
nobody |
16-1379 16 days ago |
16-1380 16 days ago |
5-11006 5 days |
| 26857 |
Thmoas-Guan author:Thmoas-Guan |
feat(Algebra): define associated graded structure for abelian group |
In this PR we define the associated graded structure for abelian group when given a filtration and only give some basic lemmas about it.
Further results would be given in #26858
---
[](https://gitpod.io/from-referrer/)
migrated from #22631
|
t-algebra
merge-conflict
awaiting-author
label:t-algebra$ |
137/0 |
Mathlib.lean,Mathlib/RingTheory/FilteredAlgebra/AssociatedGraded.lean |
2 |
22 |
['Thmoas-Guan', 'chrisflav', 'github-actions', 'mathlib4-merge-conflict-bot'] |
chrisflav assignee:chrisflav |
16-1377 16 days ago |
16-1378 16 days ago |
20-84636 20 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
merge-conflict
|
144/5 |
Mathlib/Data/PFunctor/Univariate/Basic.lean |
1 |
20 |
['alexkeizer', 'eric-wieser', 'github-actions', 'mathlib4-merge-conflict-bot', 'quangvdao'] |
eric-wieser assignee:eric-wieser |
16-1362 16 days ago |
16-1363 16 days ago |
133-25807 133 days |
| 26920 |
yuma-mizuno author:yuma-mizuno |
feat(Tactic.CategoryTheory): add associator inserting tactic |
---
[](https://gitpod.io/from-referrer/)
|
t-category-theory
t-meta
merge-conflict
WIP
|
714/0 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/CategoryTheory/Associators.lean,MathlibTest/CategoryTheory/Associators.lean |
4 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
16-1361 16 days ago |
16-1362 16 days ago |
0-16 16 seconds |
| 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
merge-conflict
|
401/0 |
Mathlib.lean,Mathlib/Dynamics/BirkhoffSum/Pointwise.lean |
2 |
14 |
['D-Thomine', 'github-actions', 'leanprover-community-bot-assistant', 'lua-vr', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
urkud assignee:urkud |
16-1359 16 days ago |
16-1360 16 days ago |
91-66923 91 days |
| 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.
---
- [x] depends on: #26836
[](https://gitpod.io/from-referrer/)
|
t-order
merge-conflict
WIP
|
238/0 |
Mathlib.lean,Mathlib/Order/Hom/Lattice.lean,Mathlib/Order/LatticeElements.lean |
3 |
5 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
16-1352 16 days ago |
16-1353 16 days ago |
0-40786 11 hours |
| 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
merge-conflict
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 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
16-1351 16 days ago |
16-1352 16 days ago |
0-45 45 seconds |
| 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
merge-conflict
awaiting-author
label:t-algebra$ |
53/0 |
Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Sheaf/VectorBundle.lean |
2 |
5 |
['Kiolt', 'Raph-DG', 'chrisflav', 'github-actions', 'mathlib4-merge-conflict-bot'] |
chrisflav assignee:chrisflav |
16-1348 16 days ago |
16-1349 16 days ago |
16-82639 16 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
merge-conflict
awaiting-author
|
1266/0 |
Mathlib.lean,Mathlib/Combinatorics/SimpleGraph/Triangle/IndependenceNumber.lean |
2 |
10 |
['Pjotr5', 'github-actions', 'grunweg', 'mathlib4-merge-conflict-bot'] |
nobody |
16-1346 16 days ago |
16-1347 16 days ago |
39-17587 39 days |
| 27163 |
pechersky author:pechersky |
feat(Topology/ValuativeRel): of and to basis of compatible valuations |
---
[](https://gitpod.io/from-referrer/)
- [x] depends on: #30262 |
t-algebra
t-topology
t-number-theory
merge-conflict
awaiting-author
label:t-algebra$ |
229/62 |
Mathlib/NumberTheory/LocalField/Basic.lean,Mathlib/Order/Filter/Bases/Basic.lean,Mathlib/Topology/Algebra/Valued/ValuativeRel.lean |
3 |
73 |
['erdOne', 'github-actions', 'kckennylau', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'pechersky', 'smmercuri'] |
alreadydone assignee:alreadydone |
16-1345 16 days ago |
16-1346 16 days ago |
86-17205 86 days |
| 27187 |
Komyyy author:Komyyy |
feat: `NONote` represents ordinals < ε₀ |
---
[](https://gitpod.io/from-referrer/)
|
t-set-theory
merge-conflict
WIP
|
186/12 |
Mathlib/SetTheory/Ordinal/Notation.lean |
1 |
3 |
['github-actions', 'mathlib4-merge-conflict-bot', 'vihdzp'] |
nobody |
16-1344 16 days ago |
16-1345 16 days ago |
0-2 2 seconds |
| 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.
---
- [x] depends on: #28614
- [x] depends on: #28615
[](https://gitpod.io/from-referrer/)
|
t-algebraic-geometry
merge-conflict
awaiting-author
|
312/0 |
Mathlib.lean,Mathlib/AlgebraicGeometry/OpenImmersion.lean,Mathlib/AlgebraicGeometry/Sites/BigAffineZariski.lean |
3 |
33 |
['chrisflav', 'github-actions', 'joelriou', 'kckennylau', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
chrisflav assignee:chrisflav |
16-1343 16 days ago |
16-1344 16 days ago |
4-4834 4 days |
| 27245 |
rirarika author:rirarika |
feat: multivariate polynomial ring properties about irreducibility |
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-algebra
merge-conflict
awaiting-author
label:t-algebra$ |
88/0 |
Mathlib.lean,Mathlib/Algebra/MvPolynomial/Irreducible.lean |
2 |
6 |
['alreadydone', 'github-actions', 'mathlib4-merge-conflict-bot', 'mbkybky'] |
alreadydone assignee:alreadydone |
16-1340 16 days ago |
16-1341 16 days ago |
109-22535 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
merge-conflict
awaiting-author
|
146/0 |
Mathlib.lean,Mathlib/Topology/Subpath.lean |
2 |
25 |
['ADedecker', 'FrankieNC', 'Sebi-Kumar', 'github-actions', 'mathlib4-merge-conflict-bot', 'themathqueen', 'wwylele'] |
ADedecker assignee:ADedecker |
16-1216 16 days ago |
16-1217 16 days ago |
34-15767 34 days |
| 27262 |
Timeroot author:Timeroot |
feat(Tactic/Bound): bound? for proof scripts |
---
[](https://gitpod.io/from-referrer/)
|
t-meta
merge-conflict
awaiting-author
|
24/9 |
Mathlib/Tactic/Bound.lean |
1 |
11 |
['JovanGerb', 'Timeroot', 'github-actions', 'j-loreaux', 'mathlib4-merge-conflict-bot'] |
nobody |
16-1215 16 days ago |
16-1216 16 days ago |
69-47369 69 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
merge-conflict
awaiting-author
|
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 |
17 |
['chrisflav', 'erdOne', 'eric-wieser', 'github-actions', 'mathlib4-merge-conflict-bot', 'ocfnash', 'xyzw12345'] |
mattrobball assignee:mattrobball |
16-1213 16 days ago |
16-1213 16 days ago |
118-9934 118 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
merge-conflict
WIP
|
218/0 |
Mathlib.lean,Mathlib/CategoryTheory/Comma/Presheaf/LeftExtension.lean |
2 |
4 |
['erdOne', 'github-actions', 'mathlib4-merge-conflict-bot', 'robin-carlier'] |
erdOne assignee:erdOne |
16-1212 16 days ago |
16-1212 16 days ago |
15-69033 15 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
merge-conflict
|
136/0 |
Mathlib.lean,Mathlib/CategoryTheory/FiberedCategory/Fiber.lean,Mathlib/CategoryTheory/Limits/Shapes/Fiberwise.lean |
3 |
25 |
['github-actions', 'kckennylau', 'mathlib4-merge-conflict-bot', 'robin-carlier'] |
nobody |
16-1210 16 days ago |
16-1211 16 days ago |
19-15685 19 days |
| 27417 |
PierreQuinton author:PierreQuinton |
feat: add `SigmaCompleteLattice` |
A $\sigma$-complete lattice is a lattice in which every countable subset `s` has a least upper bound and a greatest lower bound, denoted below by `sSup s` and `sInf s`.
This PR adds the classes `SigmaCompleteLattice` as well as some theorems (mainly adapted from `CompleteLattice` and `ConditionallyCompleteLattice`). This is an adaptation of #26318
---
[](https://gitpod.io/from-referrer/)
|
t-order
merge-conflict
awaiting-author
|
394/0 |
Mathlib.lean,Mathlib/Order/SigmaCompleteLattice.lean |
2 |
9 |
['PierreQuinton', 'YaelDillies', 'github-actions', 'mathlib4-merge-conflict-bot', 'vihdzp'] |
YaelDillies assignee:YaelDillies |
16-1207 16 days ago |
16-1208 16 days ago |
12-33338 12 days |
| 27500 |
Komyyy author:Komyyy |
feat: the Riemann zeta function is meromorphic |
Also proves that the Hurwitz zeta function is meromorphic. This PR is split from #27499 to leave a good git diff history.
---
The `large-import` change occurs only in the new module, so it poses no problem.
- [x] depends on: #27499
- [x] depends on: #29817
This PR continues the work from #25597.
Original PR: https://github.com/leanprover-community/mathlib4/pull/25597 |
large-import
t-analysis
merge-conflict
WIP
|
51/3 |
Mathlib.lean,Mathlib/Analysis/Meromorphic/Complex.lean,Mathlib/Analysis/Meromorphic/Gamma.lean |
3 |
14 |
['Komyyy', 'github-actions', 'j-loreaux', 'loefflerd', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
j-loreaux assignee:j-loreaux |
16-1203 16 days ago |
16-1204 16 days ago |
30-62878 30 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
merge-conflict
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 |
14 |
['Hagb', 'github-actions', 'grunweg', 'mathlib4-merge-conflict-bot'] |
nobody |
16-1200 16 days ago |
16-1201 16 days ago |
0-0 0 seconds |
| 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
merge-conflict
|
121/8 |
Mathlib.lean,Mathlib/Order/CompleteLattice/Defs.lean,Mathlib/Order/LawfulSupInf.lean |
3 |
26 |
['PierreQuinton', 'YaelDillies', 'github-actions', 'mathlib4-merge-conflict-bot', 'plp127', 'vihdzp'] |
YaelDillies assignee:YaelDillies |
16-1199 16 days ago |
16-1200 16 days ago |
114-58354 114 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
merge-conflict
awaiting-author
|
70/1 |
Mathlib/CategoryTheory/Category/Factorisation.lean |
1 |
13 |
['YunkaiZhang233', 'b-mehta', 'github-actions', 'mathlib4-merge-conflict-bot', 'robin-carlier'] |
nobody |
16-1191 16 days ago |
16-1192 16 days ago |
0-3448 57 minutes |
| 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
merge-conflict
awaiting-author
|
103/0 |
Mathlib.lean,Mathlib/Analysis/Calculus/Deriv/Order.lean |
2 |
37 |
['ChrisHughes24', 'EtienneC30', 'b-mehta', 'github-actions', 'j-loreaux', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'urkud'] |
hrmacbeth assignee:hrmacbeth |
16-1190 16 days ago |
16-1191 16 days ago |
85-25442 85 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
merge-conflict
awaiting-author
|
80/0 |
Mathlib.lean,Mathlib/Geometry/Manifold/ZeroDim.lean |
2 |
14 |
['fyqing', 'github-actions', 'grunweg', 'mathlib4-merge-conflict-bot', 'tb65536'] |
grunweg assignee:grunweg |
16-1189 16 days ago |
16-1190 16 days ago |
0-6418 1 hour |
| 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
merge-conflict
awaiting-author
label:t-algebra$ |
54/2 |
Mathlib/RingTheory/Ideal/Quotient/Basic.lean,Mathlib/Topology/Algebra/Valued/WithZeroMulInt.lean |
2 |
9 |
['github-actions', 'mathlib4-merge-conflict-bot', 'pechersky', 'smmercuri'] |
nobody |
16-1063 16 days ago |
16-1064 16 days ago |
44-43929 44 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
merge-conflict
WIP
|
785/0 |
Mathlib.lean,Mathlib/Geometry/Manifold/ExistsRiemannianMetric.lean,Mathlib/Geometry/Manifold/ExistsRiemannianMetric2.lean,Mathlib/Geometry/Manifold/VectorBundle/Riemannian.lean |
4 |
4 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
16-1062 16 days ago |
16-1063 16 days ago |
0-0 0 seconds |
| 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
merge-conflict
awaiting-author
|
455/13 |
Mathlib/RingTheory/Valuation/Basic.lean,MathlibTest/Simproc/ValEquiv.lean |
2 |
43 |
['b-mehta', 'erdOne', 'eric-wieser', 'github-actions', 'kckennylau', 'mathlib4-merge-conflict-bot', 'pechersky', 'plp127'] |
erdOne assignee:erdOne |
16-1061 16 days ago |
16-1061 16 days ago |
99-49574 99 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
merge-conflict
|
79/0 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Simproc/Apply.lean,MathlibTest/Simproc/Apply.lean |
4 |
28 |
['JovanGerb', 'b-mehta', 'eric-wieser', 'github-actions', 'hrmacbeth', 'kckennylau', 'mathlib4-merge-conflict-bot'] |
JovanGerb assignee:JovanGerb |
16-1058 16 days ago |
16-1059 16 days ago |
93-19048 93 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
merge-conflict
|
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 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
awainverse assignee:awainverse |
16-1057 16 days ago |
16-1058 16 days ago |
102-43516 102 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
merge-conflict
awaiting-author
|
16/0 |
Mathlib/Tactic/FunProp.lean |
1 |
6 |
['Vierkantor', 'github-actions', 'grunweg', 'kckennylau', 'mathlib4-merge-conflict-bot'] |
alexjbest assignee:alexjbest |
16-1056 16 days ago |
16-1057 16 days ago |
57-63332 57 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
merge-conflict
|
136/5 |
Mathlib.lean,Mathlib/Tactic/NormNum/Core.lean,Mathlib/Util/Trace.lean,MathlibTest/norm_num_trace.lean |
4 |
20 |
['JovanGerb', 'eric-wieser', 'github-actions', 'kmill', 'leanprover-bot', 'mathlib-bors', 'mathlib4-merge-conflict-bot', 'plp127'] |
JovanGerb assignee:JovanGerb |
16-1051 16 days ago |
16-1052 16 days ago |
98-33060 98 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
merge-conflict
|
81/2 |
Mathlib/Topology/Algebra/GroupWithZero.lean,Mathlib/Topology/Algebra/WithZeroTopology.lean,Mathlib/Topology/Compactness/Compact.lean |
3 |
13 |
['erdOne', 'github-actions', 'kckennylau', 'mathlib4-merge-conflict-bot', 'ocfnash'] |
PatrickMassot assignee:PatrickMassot |
16-1050 16 days ago |
16-1051 16 days ago |
98-8139 98 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 "[" "]" Polynomial Polynomial.C Polynomial.X
register_poly_vars (mv := true) "[" "]" 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 be valid syntax.
There has been some discussion about its implementation:
* It has been suggested that `R[x,y][z]` should mean that `R[x,y]` is a subring, i.e. `x` should live in `R[x,y]`, but in my implementation `x` lives in the big ring `R[x,y][z]`. There are two ways to get the other behaviour:
* One can do `R[x,y]` and then `(R[x,y])[z]`.
* One can do `R[a,b]` and `R[x,y][z]`. I personally prefer this one because we should make it clearer that they are different rings.
* There has been some discussion over what `R` means. In my implementation, if you ever refer to a `variable` called `R`, then `R` is fixed to that variable, meaning that if you later define a variable with the same name, `R` will still refer to the old variable. Also, this does not respect namespace, meaning that if you refer to `Foo.bar[x,y]`, and later open `Foo`, you will not be able to access the declared ring with `bar[x,y]`.
---
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)
This is a refactor of the currently existing [Mathlib.Tactic.namePolyVarsOver](https://leanprover-community.github.io/mathlib4_docs/Mathlib/Tactic/Ring/NamePolyVars.html#Mathlib.Tactic.namePolyVarsOver). More explicitly, the current invocation `name_poly_vars x,y over R` is now `poly_variable R[x,y]`. The behaviours inherited from `name_poly_vars` are:
* We do not synthesize the necessary instances (such as `[CommRing R]`) at the point of declaration, but only when the new notations are used.
* We refer to an explicit term (`R` in the examples) which is "fixed", in the sense that:
* it is only valid for `R` explicitly, and not any other `variable` such as `S`.
* it has built-in hygiene, so if you shadow the variable by declaring a new `variable (R : Type*)`, it will still refer to the old one.
And the new behaviours are:
* Currently only `x` and `y` are new notations, but in the new tactic the whole ring `R[x,y]` is also available as notation.
* Currently only the forward direction (i.e. elaboration, going from `x` to `MvPolynomial.X 0`) is implemented, but in the new tactic we also implement the backward direction, printing `MvPolynomial.X 0` back as `x` (and `MvPolynomial (Fin 2) R` is printed as `R[x,y]`).
* Support beyond just `MvPolynomial`.
* Support for nested polynomial-like rings, such as `R[x,y][t][[z]]` for `PowerSeries (Polynomial (MvPolynomial (Fin 2) R))`.
[](https://gitpod.io/from-referrer/)
|
t-meta
merge-conflict
awaiting-author
|
778/87 |
Counterexamples/CliffordAlgebraNotInjective.lean,Mathlib.lean,Mathlib/Algebra/MvPolynomial/Basic.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Jacobian/Basic.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Projective/Basic.lean,Mathlib/Tactic.lean,Mathlib/Tactic/PolyVariable.lean,Mathlib/Tactic/Ring/NamePolyVars.lean,MathlibTest/PolyVariable.lean,scripts/noshake.json |
10 |
110 |
['JovanGerb', 'adamtopaz', 'chrisflav', 'eric-wieser', 'github-actions', 'j-loreaux', 'kckennylau', 'kim-em', 'mathlib4-merge-conflict-bot', 'plp127', 'robertmaxton42', 'sgouezel'] |
adamtopaz assignee:adamtopaz |
16-1047 16 days ago |
16-1048 16 days ago |
69-30520 69 days |
| 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
merge-conflict
label:t-algebra$ |
41/13 |
Mathlib/Algebra/Order/Positive/Field.lean,Mathlib/Algebra/Order/Positive/Ring.lean,Mathlib/Data/PNat/Defs.lean |
3 |
3 |
['github-actions', 'mathlib4-merge-conflict-bot', 'yury-harmonic'] |
nobody |
16-905 16 days ago |
16-906 16 days ago |
86-47209 86 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
merge-conflict
|
62/0 |
Mathlib.lean,Mathlib/Combinatorics/Digraph/Orientation.lean,Mathlib/Combinatorics/Digraph/Tournament.lean |
3 |
6 |
['JaafarTanoukhi', 'Rida-Hamadani', 'SnirBroshi', 'github-actions', 'mathlib4-merge-conflict-bot'] |
kmill assignee:kmill |
16-904 16 days ago |
16-905 16 days ago |
86-45080 86 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
merge-conflict
awaiting-author
|
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 |
9 |
['github-actions', 'kckennylau', 'mathlib4-merge-conflict-bot'] |
alreadydone assignee:alreadydone |
16-900 16 days ago |
16-901 16 days ago |
71-25577 71 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
merge-conflict
awaiting-author
|
91/0 |
Mathlib.lean,Mathlib/MeasureTheory/Function/LInfty.lean |
2 |
6 |
['JonBannon', 'github-actions', 'j-loreaux', 'mathlib4-merge-conflict-bot'] |
nobody |
16-897 16 days ago |
16-898 16 days ago |
4-12126 4 days |
| 29235 |
yoh-tanimoto author:yoh-tanimoto |
feat(Topology/Algebra/Module/ClosedSubmodule): add `mapEquiv`, a variation of `ClosedSubmodule.map` for CLE |
add `ClosedSubmodule.mapEquiv` for continuous linear equivalence. In this case, a closed submodule is mapped to a closed submodule, 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
merge-conflict
|
69/1 |
Mathlib/Topology/Algebra/Module/ClosedSubmodule.lean |
1 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
fpvandoorn assignee:fpvandoorn |
16-890 16 days ago |
16-891 16 days ago |
67-57008 67 days |
| 29411 |
llllvvuu author:llllvvuu |
feat(LinearAlgebra/Matrix/Rank): rank factorization |
The rank factorization derived from `Module.finBasis`.
Co-authored-by: Aristotle Harmonic
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict
awaiting-author
|
20/0 |
Mathlib/LinearAlgebra/Matrix/Rank.lean,Mathlib/LinearAlgebra/Matrix/ToLin.lean |
2 |
3 |
['github-actions', 'jcommelin', 'mathlib4-merge-conflict-bot'] |
jcommelin assignee:jcommelin |
16-878 16 days ago |
16-879 16 days ago |
46-58434 46 days |
| 29481 |
llllvvuu author:llllvvuu |
feat(LinearAlgebra/Eigenspace): roots of matrix minpoly give spectrum |
This is derived from the corresponding result on linear maps.
---
- [x] depends on: #29478 for some simp lemmas
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebra
merge-conflict
label:t-algebra$ |
13/0 |
Mathlib/LinearAlgebra/Eigenspace/Minpoly.lean |
1 |
5 |
['github-actions', 'llllvvuu', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
16-872 16 days ago |
16-872 16 days ago |
0-0 0 seconds |
| 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
merge-conflict
awaiting-author
|
31/0 |
Mathlib.lean,Mathlib/Order/UpperLower/WellFounded.lean |
2 |
3 |
['github-actions', 'mathlib4-merge-conflict-bot', 'plp127'] |
bryangingechen assignee:bryangingechen |
16-870 16 days ago |
16-871 16 days ago |
10-85553 10 days |
| 29526 |
llllvvuu author:llllvvuu |
feat: `Multiset.map f` identifies `f` up to permutation |
Motivation: Reason about `Fintype`-indexed families via `Multiset` equality.
Example use case 1:
```lean
theorem Matrix.IsHermitian.cfc_eigenvalues {d : Type*} [Fintype d] [DecidableEq d]
{M : Matrix d d 𝕜} (hM : M.IsHermitian) (f : ℝ → ℝ)
(hcfc : Matrix.IsHermitian (cfc f M) := cfc_predicate f M) :
∃ (e : d ≃ d), hcfc.eigenvalues = f ∘ hM.eigenvalues ∘ e := by
have := hcfc.roots_charpoly_eq_eigenvalues.symm
rw [hM.charpoly_cfc_eq f, Polynomial.roots_prod] at this; swap
· simp [Finset.prod_ne_zero_iff, Polynomial.X_sub_C_ne_zero]
simp_rw [Polynomial.roots_X_sub_C, Multiset.bind_singleton] at this
have he := (Multiset.compTriple_equivOfMapUnivEq this).comp_eq
simp_rw [← Function.comp_def RCLike.ofReal, ← Function.comp_def f, Function.comp_assoc] at he
exact ⟨_, RCLike.ofReal_injective.comp_left he.symm⟩
```
Example use case 2 (on top of https://github.com/leanprover-community/mathlib4/pull/29610):
```lean
theorem LinearMap.Eigenbasis.μ_equiv {ι ι' R G : Type*} [Fintype ι] [Fintype ι']
[CommRing R] [IsDomain R] [AddCommGroup G] [Module R G] [Module.Free R G] [Module.Finite R G]
{f : Module.End R G} (B₁ : f.Eigenbasis ι) (B₂ : f.Eigenbasis ι') :
∃ e : ι ≃ ι', B₁.μ = B₂.μ ∘ e := by
classical
have := congr(Polynomial.roots $(B₁.charpoly_eq.symm.trans B₂.charpoly_eq))
rw [Polynomial.roots_prod, Polynomial.roots_prod] at this; rotate_left
· simp [Finset.prod_ne_zero_iff, Polynomial.X_sub_C_ne_zero]
· simp [Finset.prod_ne_zero_iff, Polynomial.X_sub_C_ne_zero]
simp_rw [Polynomial.roots_X_sub_C, Multiset.bind_singleton] at this
exact ⟨Multiset.equivOfMapUnivEq this, (Multiset.compTriple_equivOfMapUnivEq this).comp_eq.symm⟩
```
Co-authored-by: Aristotle Harmonic
---
[](https://gitpod.io/from-referrer/)
|
t-data
merge-conflict
|
35/0 |
Mathlib/Data/Multiset/Fintype.lean |
1 |
9 |
['Ruben-VandeVelde', 'github-actions', 'llllvvuu', 'mathlib4-merge-conflict-bot', 'vihdzp', 'wwylele'] |
pechersky assignee:pechersky |
16-866 16 days ago |
16-867 16 days ago |
69-23592 69 days |
| 29610 |
llllvvuu author:llllvvuu |
feat(LinearAlgebra): define LinearMap.Eigenbasis |
Some theorems are left TODO for follow-up work.
The definition is from @eric-wieser ([#Is there code for X? > diagonalizable linear maps @ 💬](https://leanprover.zulipchat.com/#narrow/channel/217875-Is-there-code-for-X.3F/topic/diagonalizable.20linear.20maps/near/539163222)).
Co-authored-by: Aristotle Harmonic
---
- [x] depends on: #29420 (golfs some `[Nontrivial R]` assumptions)
- [x] depends on: #29791
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
label:t-algebra$ |
455/5 |
Mathlib.lean,Mathlib/Analysis/InnerProductSpace/Spectrum.lean,Mathlib/LinearAlgebra/Eigenbasis.lean,Mathlib/LinearAlgebra/FreeModule/PID.lean,Mathlib/Order/CompleteLattice/Basic.lean |
5 |
30 |
['github-actions', 'kckennylau', 'llllvvuu', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
joelriou assignee:joelriou |
16-301 16 days ago |
16-302 16 days ago |
22-46437 22 days |
| 29675 |
yury-harmonic author:yury-harmonic |
feat(Wolstenholme): new file |
Co-authored-by: @Aristotle-Harmonic
---
I still need to cleanup the proof and write the docs.
For now, it's just what the AI generated, forward-ported to the latest Mathlib.
[](https://gitpod.io/from-referrer/)
|
t-data
merge-conflict
awaiting-author
help-wanted
|
198/0 |
Mathlib.lean,Mathlib/Data/Nat/Choose/Wolstenholme.lean |
2 |
4 |
['github-actions', 'mathlib4-merge-conflict-bot', 'yury-harmonic'] |
nobody |
16-295 16 days ago |
16-296 16 days ago |
0-125 2 minutes |
| 29720 |
javra author:javra |
feat(CategoryTheory): `TransportEnrichment` and `ForgetEnrichment` as 2-functors |
---
[](https://gitpod.io/from-referrer/)
|
t-category-theory
merge-conflict
WIP
|
63/1 |
Mathlib/CategoryTheory/Enriched/Basic.lean,Mathlib/CategoryTheory/Enriched/EnrichedCat.lean |
2 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
16-288 16 days ago |
16-288 16 days ago |
0-24 24 seconds |
| 29827 |
js2357 author:js2357 |
feat: define two (trivial) ContinuousMulEquivs |
Define two trivial `ContinuousMulEquiv`s:
`ContinuousMulEquiv.piUnique` is the topological version of `MulEquiv.piUnique`.
`ContinuousMulEquiv.piEquivPiSubtypeProd` is the multiplicative version of `Homeomorph.piEquivPiSubtypeProd`.
Done for the FLT project.
---
[](https://gitpod.io/from-referrer/)
|
large-import
FLT
t-topology
merge-conflict
|
25/0 |
Mathlib/Topology/Algebra/ContinuousMonoidHom.lean |
1 |
3 |
['github-actions', 'grunweg', 'mathlib4-merge-conflict-bot'] |
nobody |
16-274 16 days ago |
16-275 16 days ago |
60-20058 60 days |
| 29947 |
JaafarTanoukhi author:JaafarTanoukhi |
feat(Combinatorics/Digraph): Maps |
Ported `SimpleGraph/Maps.lean` to `Digraph/Maps.lean` for future PRs related to issue #[26771](https://github.com/leanprover-community/mathlib4/issues/26771)
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-combinatorics
merge-conflict
|
476/0 |
Mathlib.lean,Mathlib/Combinatorics/Digraph/Maps.lean |
2 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
awainverse assignee:awainverse |
16-270 16 days ago |
16-271 16 days ago |
55-55764 55 days |
| 29965 |
RemyDegenne author:RemyDegenne |
feat(probability): define subtraction of kernels |
This PR defines subtraction of kernels and uses it to prove `MeasurableSet {a | κ a = η a}` for two finite kernels `κ, η`.
From the LeanBandits project.
---
[](https://gitpod.io/from-referrer/)
|
t-measure-probability
merge-conflict
WIP
|
288/1 |
Mathlib.lean,Mathlib/MeasureTheory/Measure/Sub.lean,Mathlib/MeasureTheory/Measure/SubFinite.lean,Mathlib/Probability/Kernel/Defs.lean,Mathlib/Probability/Kernel/RadonNikodym.lean,Mathlib/Probability/Kernel/Sub.lean |
6 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
16-266 16 days ago |
16-267 16 days ago |
0-1 1 second |
| 29980 |
mans0954 author:mans0954 |
refactor(RingTheory/Polynomial/Resultant/Quadratic): Re-implement QuadraticDiscriminant for R[X] |
Re-implement `Algebra/QuadraticDiscriminant` for polynomials.
[Zulip discussion](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/discriminants.20of.20low.20degree.20polynomials/with/538010519)
---
- [ ] depends on: #29981
[](https://gitpod.io/from-referrer/)
|
merge-conflict |
208/0 |
Mathlib.lean,Mathlib/RingTheory/Polynomial/Resultant/Quadratic.lean |
2 |
4 |
['JovanGerb', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
JovanGerb assignee:JovanGerb |
16-263 16 days ago |
16-264 16 days ago |
41-49356 41 days |
| 30004 |
luigi-massacci author:luigi-massacci |
feat(MeasureTheory/Integral/TestAgainst): integrating BCFs against a finite measure or an L1Loc map as CLMs |
This PR merges #29511 and #29748. Create a new file `TestAgainst.lean` with definitions wrapping integration against a finite measure or a locally integrable map as continuous linear maps on bounded continuous functions.
---
[](https://gitpod.io/from-referrer/)
|
t-measure-probability
t-analysis
merge-conflict
awaiting-author
|
112/1 |
Mathlib.lean,Mathlib/MeasureTheory/Integral/BoundedContinuousFunction.lean,Mathlib/MeasureTheory/Integral/TestAgainst.lean |
3 |
48 |
['EtienneC30', 'github-actions', 'j-loreaux', 'luigi-massacci', 'mathlib4-merge-conflict-bot'] |
EtienneC30 assignee:EtienneC30 |
16-257 16 days ago |
16-258 16 days ago |
31-80552 31 days |
| 30022 |
ADedecker author:ADedecker |
feat: theory of `IsRightUniformGroup` and `IsLeftUniformGroup` |
---
[](https://gitpod.io/from-referrer/)
|
t-topology
merge-conflict
|
799/150 |
Mathlib/Topology/Algebra/IsUniformGroup/Basic.lean,Mathlib/Topology/Algebra/IsUniformGroup/Defs.lean |
2 |
7 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
16-256 16 days ago |
16-257 16 days ago |
0-0 0 seconds |
| 30042 |
JovanGerb author:JovanGerb |
feat(push): `@[push]` attributes for `∈` in `Set`, `Finset` and `Multiset` |
This PR adds `@[push]` annotations for the membership relations, for `Set`, `Finset` and `Multiset`.
---
[](https://gitpod.io/from-referrer/)
|
t-meta
merge-conflict
awaiting-author
|
171/105 |
Mathlib/Algebra/BigOperators/Group/Finset/Basic.lean,Mathlib/Algebra/Group/Pointwise/Finset/Basic.lean,Mathlib/Algebra/Group/Pointwise/Set/Basic.lean,Mathlib/Algebra/Group/Pointwise/Set/ListOfFn.lean,Mathlib/Algebra/Order/Group/Multiset.lean,Mathlib/Data/DFinsupp/Interval.lean,Mathlib/Data/Finmap.lean,Mathlib/Data/Finset/BooleanAlgebra.lean,Mathlib/Data/Finset/Dedup.lean,Mathlib/Data/Finset/Defs.lean,Mathlib/Data/Finset/Disjoint.lean,Mathlib/Data/Finset/Filter.lean,Mathlib/Data/Finset/Image.lean,Mathlib/Data/Finset/Insert.lean,Mathlib/Data/Finset/Lattice/Basic.lean,Mathlib/Data/Finset/Lattice/Fold.lean,Mathlib/Data/Finset/Pi.lean,Mathlib/Data/Finset/Powerset.lean,Mathlib/Data/Finset/Range.lean,Mathlib/Data/Finset/SDiff.lean,Mathlib/Data/Finset/Sigma.lean,Mathlib/Data/Finset/Sort.lean,Mathlib/Data/Finset/Sum.lean,Mathlib/Data/Finset/Sups.lean,Mathlib/Data/Finset/Union.lean,Mathlib/Data/Fintype/Defs.lean,Mathlib/Data/Multiset/AddSub.lean,Mathlib/Data/Multiset/Antidiagonal.lean,Mathlib/Data/Multiset/Bind.lean,Mathlib/Data/Multiset/Dedup.lean,Mathlib/Data/Multiset/Defs.lean,Mathlib/Data/Multiset/Filter.lean,Mathlib/Data/Multiset/FinsetOps.lean,Mathlib/Data/Multiset/MapFold.lean,Mathlib/Data/Multiset/Pi.lean,Mathlib/Data/Multiset/Range.lean,Mathlib/Data/Multiset/Replicate.lean,Mathlib/Data/Multiset/Sort.lean,Mathlib/Data/Multiset/Sum.lean,Mathlib/Data/Multiset/UnionInter.lean,Mathlib/Data/Multiset/ZeroCons.lean,Mathlib/Data/Set/Basic.lean,Mathlib/Data/Set/Insert.lean,Mathlib/Data/Set/Operations.lean,Mathlib/Order/Interval/Finset/Defs.lean,Mathlib/Order/Interval/Multiset.lean,Mathlib/Order/Interval/Set/Defs.lean,Mathlib/Order/SetNotation.lean,MathlibTest/push.lean |
49 |
14 |
['JovanGerb', 'github-actions', 'grunweg', 'mathlib4-merge-conflict-bot'] |
grunweg assignee:grunweg |
16-251 16 days ago |
16-252 16 days ago |
23-81049 23 days |
| 30105 |
slashbade author:slashbade |
feat: add `reap` as internal tactic |
---
[](https://gitpod.io/from-referrer/)
|
large-import
new-contributor
t-meta
merge-conflict
|
664/0 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Common.lean,Mathlib/Tactic/Reap.lean,Mathlib/Tactic/Reap/Basic.lean,Mathlib/Tactic/Reap/Future/Basic.lean,Mathlib/Tactic/Reap/Future/PP.lean,Mathlib/Tactic/Reap/OpenAIClient/Basic.lean,Mathlib/Tactic/Reap/OpenAIClient/Test.lean,Mathlib/Tactic/Reap/OpenAIClient/Types.lean,Mathlib/Tactic/Reap/Options.lean,Mathlib/Tactic/Reap/PremiseSelection/API.lean,Mathlib/Tactic/Reap/PremiseSelection/Syntax.lean,Mathlib/Tactic/Reap/PremiseSelection/Test.lean,Mathlib/Tactic/Reap/Requests/Basic.lean,Mathlib/Tactic/Reap/Requests/Future.lean,Mathlib/Tactic/Reap/Requests/Test.lean,Mathlib/Tactic/Reap/Tactic/Generator.lean,Mathlib/Tactic/Reap/Tactic/Search.lean,Mathlib/Tactic/Reap/Tactic/Syntax.lean,Mathlib/Tactic/Reap/Tactic/Test.lean |
21 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
16-242 16 days ago |
16-243 16 days ago |
0-0 0 seconds |
| 30121 |
idontgetoutmuch author:idontgetoutmuch |
Principal fiber bundle core |
A structure capturing what it means to be a principal fibre bundle.
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-differential-geometry
merge-conflict
awaiting-author
|
227/0 |
Mathlib.lean,Mathlib/Geometry/Manifold/PrincipalFiberBundle/PrincipalGBundle.lean |
2 |
6 |
['github-actions', 'grunweg', 'mathlib4-merge-conflict-bot'] |
hrmacbeth assignee:hrmacbeth |
16-237 16 days ago |
16-238 16 days ago |
25-22983 25 days |
| 30131 |
fpvandoorn author:fpvandoorn |
feat: alias_in attribute |
* A small wrapper for adding an alias of a declaration in another namespace.
* application time `.afterCompilation` is necessary for `#eval` to work correctly
* Docstrings are copied, jump-to-definition works (no test in the test file, but tested locally)
* To be used for CW-complexes, where lemmas are frequently duplicated between `RelCWComplex` and `CWComplex`.
---
[](https://gitpod.io/from-referrer/)
cc @scholzhannah
|
t-meta
merge-conflict
|
93/0 |
Mathlib.lean,Mathlib/Util/AliasIn.lean,MathlibTest/Util/AliasIn.lean |
3 |
14 |
['JovanGerb', 'fpvandoorn', 'github-actions', 'mathlib4-merge-conflict-bot'] |
JovanGerb assignee:JovanGerb |
16-235 16 days ago |
16-235 16 days ago |
47-55790 47 days |
| 30233 |
Komyyy author:Komyyy |
refactor(Topology/Sequences): generalize seq-compactness lemmas to metrizable space |
* [`IsSeqCompact.isCompact`](https://leanprover-community.github.io/mathlib4_docs/Mathlib/Topology/Sequences.html#IsSeqCompact.isCompact)
* [`UniformSpace.isCompact_iff_isSeqCompact`](https://leanprover-community.github.io/mathlib4_docs/Mathlib/Topology/Sequences.html#UniformSpace.isCompact_iff_isSeqCompact)
* [`UniformSpace.compactSpace_iff_seqCompactSpace`](https://leanprover-community.github.io/mathlib4_docs/Mathlib/Topology/Sequences.html#UniformSpace.compactSpace_iff_seqCompactSpace)
These are lemmas on uniform spaces which has countable uniformity, so can be generalized to pseudo-metrizable space.
From [CLT](https://github.com/RemyDegenne/CLT)
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-topology
merge-conflict
|
20/7 |
Mathlib/Topology/Sequences.lean,docs/overview.yaml,docs/undergrad.yaml |
3 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
grunweg assignee:grunweg |
16-100 16 days ago |
16-101 16 days ago |
41-80880 41 days |
| 30330 |
Bergschaf author:Bergschaf |
feat(Algebra/Group/Action/Equidecomp): Mathlib's definition of Equidecomposability is equivalent to the standart one using partitions |
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebra
merge-conflict
label:t-algebra$ |
329/1 |
Mathlib/Algebra/Group/Action/Equidecomp.lean |
1 |
6 |
['Bergschaf', 'Felix-Weilacher', 'github-actions', 'mathlib4-merge-conflict-bot'] |
Vierkantor assignee:Vierkantor |
16-93 16 days ago |
16-94 16 days ago |
0-0 0 seconds |
| 30355 |
kckennylau author:kckennylau |
feat(Logic): graded functions |
This PR defines a class of graded functions, called `GradedFunLike`. It is intended to be used in #30312 to characterise a class of graded ring homomorphisms, where it is invoked as `[GradedFunLike F 𝒜 ℬ] [RingHomClass F A B]`.
---
[](https://gitpod.io/from-referrer/)
|
t-data
merge-conflict
|
41/0 |
Mathlib.lean,Mathlib/Data/FunLike/Graded.lean |
2 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
16-82 16 days ago |
16-83 16 days ago |
41-25826 41 days |
| 30392 |
urkud author:urkud |
feat: define pullback quotient maps |
---
[](https://gitpod.io/from-referrer/)
|
t-topology
merge-conflict
|
287/0 |
Mathlib.lean,Mathlib/Topology/ClusterPt.lean,Mathlib/Topology/Maps/PullbackQuotient.lean |
3 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
16-69 16 days ago |
16-70 16 days ago |
0-0 0 seconds |
| 30451 |
kckennylau author:kckennylau |
feat(HomogeneousIdeal): generalize to homogeneous submodule |
Continuation of #30437 with permission from @jjaassoonn, which is a continuation of #9820 .
The definitions, constructions and theorems in `HomogeneousIdeal.lean` are generalized to homogeneous submodules.
Let `R` be a graded ring and `M` be a graded `R`-module. Say an `R`-submodule `N` of `M` is homogeneous if for every `x` in `N`, each projection of `x` to `M_i` is in `N`. None of this file's results depends on the grading on `R`, but we include the grading on `R` for technical reasons. We define the "homogeneous core" of a not necessarily homogeneous submodule N to be the biggest homogeneous submodule contained within N, and the "homogeneous hull" to be the smallest homogeneous submodule that contains N.
All definitions/constructions/theorems are then copied for ideals/homogeneous ideals.
The motivation of this generalization is graded quotient module. (#18716)
---
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
merge-conflict
|
553/181 |
Mathlib/Algebra/Module/GradedModule.lean,Mathlib/AlgebraicGeometry/ProjectiveSpectrum/Basic.lean,Mathlib/AlgebraicGeometry/ProjectiveSpectrum/Scheme.lean,Mathlib/RingTheory/GradedAlgebra/Homogeneous/Ideal.lean,Mathlib/RingTheory/GradedAlgebra/Homogeneous/Submodule.lean,Mathlib/RingTheory/GradedAlgebra/Radical.lean |
6 |
3 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
mariainesdff assignee:mariainesdff |
16-67 16 days ago |
16-68 16 days ago |
23-22490 23 days |
| 30668 |
astrainfinita author:astrainfinita |
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.
This PR also adds some typeclasses to support different ways to find the quotient map that should be used. See the documentation comments of these typeclasses for examples of usage.
---
It's not a typical design to use these auxiliary typeclasses and term elaborators, but I haven't found a better way to support these notations.
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.
- It would be helpful if the names of new type classes explained their functionality better.
- Maybe `QuotLike` isn't the appropriate name. It may suggest that this typeclass is similar to `FunLike` and `SetLike`, but it is not.
[Zulip](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/migrate.20to.20.60QuotLike.60.20API)
This PR continues the work from #16421.
Original PR: https://github.com/leanprover-community/mathlib4/pull/16421 |
t-data
awaiting-zulip
RFC
merge-conflict
awaiting-author
|
743/0 |
Mathlib.lean,Mathlib/Data/QuotLike.lean,MathlibTest/QuotLike.lean |
3 |
15 |
['YaelDillies', 'astrainfinita', 'github-actions', 'mathlib4-merge-conflict-bot', 'vihdzp'] |
nobody |
15-86319 15 days ago |
15-86320 15 days ago |
0-81 1 minute |
| 30933 |
joelriou author:joelriou |
feat(CategoryTheory): the linearization of a category |
Let `C` be a category and `R` be a commutative ring. We construct a `R`-linear category `Linearization C R` and
a functor `toLinearization C R : C ⥤ Linearization C R`. The morphisms in `Linearization C R` are the free `R`-modules
on the types of morphisms in `C`.
(In the context of singular homology with coefficients `R`, chains of a fixed degree shall identify to morphisms in `Linearization TopCat R`, and doing certain computations for arbitrary coefficients should reduce to computations with `R := ℤ`.)
---
[](https://gitpod.io/from-referrer/)
|
t-category-theory
merge-conflict
awaiting-author
|
134/0 |
Mathlib.lean,Mathlib/CategoryTheory/Linear/Linearization.lean |
2 |
4 |
['github-actions', 'joelriou', 'kim-em', 'mathlib4-merge-conflict-bot'] |
nobody |
15-86161 15 days ago |
15-86162 15 days ago |
2-33570 2 days |
| 31008 |
RemyDegenne author:RemyDegenne |
refactor: generalize the index of the process in the Doob decomposition |
Generalize the index set for the Doob decomposition of an adapted process from Nat to a type with `LinearOrder`, `LocallyFiniteOrder`, `OrderBot`, `SuccOrder` (there is an order iso from that type to an interval of Nat).
Motivation: to prove the Doob-Meyer decomposition we want to take a process indexed by [0,1] and consider sub-processes indexed by the dyadic points k*2^{-n} for a fixed n. We could use a process indexed by Nat, but we would have to invent values for k > 2^n while respecting the other properties of the process, and being able to index by the dyadics directly seems easier.
---
[](https://gitpod.io/from-referrer/)
|
t-measure-probability
merge-conflict
WIP
|
295/124 |
Mathlib/Order/SuccPred/LinearLocallyFinite.lean,Mathlib/Probability/Martingale/Basic.lean,Mathlib/Probability/Martingale/BorelCantelli.lean,Mathlib/Probability/Martingale/Centering.lean,Mathlib/Probability/Martingale/OptionalStopping.lean,Mathlib/Probability/Martingale/Upcrossing.lean,Mathlib/Probability/Process/Adapted.lean |
7 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
15-86140 15 days ago |
15-86141 15 days ago |
0-2 2 seconds |
| 31102 |
JOSHCLUNE author:JOSHCLUNE |
Require LeanHammer |
Experimenting with adding LeanHammer as a mathlib dependency
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
merge-conflict
|
61/4 |
Mathlib/Tactic/Common.lean,Mathlib/Tactic/Linter/DirectoryDependency.lean,MathlibTest/Hammer.lean,lake-manifest.json,lakefile.lean |
5 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
15-86127 15 days ago |
15-86128 15 days ago |
19-46677 19 days |
| 31194 |
grunweg author:grunweg |
feat: add `#check'` command and tactic, which only show explicit arguments |
In some areas (such as differential geometry), many lemmas have a *lot* of implicit and typeclass arguments.
Using `#check foo` to determine which explicit arguments are expected for a given lemma gives output which is painful to read, because the explicit argument is buried among many lines of other output.
The `#check'` command and tactic produce very similar output, but with implicit and typeclass arguments omitted.
This increases usability a lot.
In the future, this could (and should) be unified to the #check command in core, by becoming e.g. `#check +only-explicit`. Until then, let us add this to mathlib to facilitate experimentation of the most useful behaviour.
From the project towards geodesics and the Levi-Civita connection.
Co-authored-by: Kyle Miller
Co-authored-by: Patrick Massot
---
[](https://gitpod.io/from-referrer/)
|
t-meta
merge-conflict
awaiting-author
|
151/11 |
Mathlib/Tactic/Check.lean,MathlibTest/Check.lean |
2 |
12 |
['github-actions', 'grunweg', 'mathlib4-merge-conflict-bot', 'thorimur'] |
thorimur assignee:thorimur |
15-86102 15 days ago |
15-86103 15 days ago |
12-18469 12 days |
| 31314 |
hrmacbeth author:hrmacbeth |
feat: linters for recommended `field_simp` style |
---
- [x] depends on: #31472
- [x] depends on: #31483
[](https://gitpod.io/from-referrer/)
|
t-linter
awaiting-CI
merge-conflict
|
93/1 |
Mathlib.lean,Mathlib/Lean/Meta/WarningAsError.lean,Mathlib/Tactic/Field.lean |
3 |
5 |
['github-actions', 'grunweg', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
15-85961 15 days ago |
15-85961 15 days ago |
0-0 0 seconds |
| 31351 |
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: #30049 (preliminary code clean-up)
- [x] depends on: #29589
- [x] ~~depends on: https://github.com/grunweg/mathlib4/tree/mfderiv-prodmap for actually proving the mfderiv sorry about products I need~~ done now
- [ ] depends on: #31200 (and its companion result, about Sum.map)
- [ ] depends on #23040 for the mathlib-level definition of smooth immersions and embeddings
This PR continues the work from #22059.
---
[](https://gitpod.io/from-referrer/)
|
t-differential-geometry
merge-conflict
WIP
|
591/0 |
Mathlib.lean,Mathlib/Geometry/Manifold/HasSmoothBoundary.lean |
2 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
15-85735 15 days ago |
15-85735 15 days ago |
0-13 13 seconds |
| 31356 |
adomani author:adomani |
feat: add inspect-like functions |
Produces a tree-like formatting for `Syntax`, `Expr` and `InfoTree`. Especially for the `InfoTree`s, there are *many* parts of it that do not get printed.
For instance, this is how the `InfoTree`s of `set_option linter.missingDocs true` get printed:
```lean
inspectIT
set_option linter.missingDocs true
/-
commandCtx
|-Info.ofCommandInfo: Lean.Elab.Command.elabSetOption, 'set_option…gDocs true'
| |-Info.ofCompletionInfo.CompletionInfo.option 'set_option…issingDocs'
| |-Info.ofOptionInfo: linter.missingDocs, Linter.linter.missingDocs
-/
```
---
[](https://gitpod.io/from-referrer/)
|
t-meta
merge-conflict
|
720/0 |
Mathlib.lean,Mathlib/Util/Inspect.lean,MathlibTest/Inspect.lean |
3 |
3 |
['github-actions', 'mathlib4-merge-conflict-bot', 'plp127'] |
kim-em assignee:kim-em |
15-81691 15 days ago |
15-81692 15 days ago |
11-75498 11 days |
| 31604 |
maksym-radziwill author:maksym-radziwill |
feat: analyticity of dslope |
This adds a few simple functions to show that ``dslope f a`` is analytic when ``f`` is. This is needed for Borel-Caratheodory, see https://github.com/leanprover-community/mathlib4/pull/30424
---
[](https://gitpod.io/from-referrer/)
|
t-analysis
merge-conflict
awaiting-author
|
51/0 |
Mathlib.lean,Mathlib/Analysis/Analytic/Dslope.lean |
2 |
26 |
['github-actions', 'grunweg', 'maksym-radziwill', 'mathlib4-merge-conflict-bot'] |
nobody |
15-81395 15 days ago |
15-81396 15 days ago |
0-3879 1 hour |
| 31613 |
xyzw12345 author:xyzw12345 |
feat(RepresentationTheory/GroupCohomology): Non-abelian Group Cohomology |
In this PR, we develop the theory of non-abelian group cohomology, following the section in GTM 67 - Local Fields by Jean-Pierre Serre. We defined H0 and H1, constructed the connection maps, proved the long exact sequence, and constructed natural isomorphisms between our H0, H1 and the existing `groupCohomology` API.
Co-authored by:
Jiedong Jiang @jjdishere
(information of other co-authors will be updated here soon)
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebra
merge-conflict
WIP
label:t-algebra$ |
406/0 |
Mathlib.lean,Mathlib/Algebra/Category/Grp/Zero.lean,Mathlib/GroupTheory/Subgroup/Center.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/NonAbelian.lean,Mathlib/RepresentationTheory/Rep.lean |
5 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
15-81391 15 days ago |
15-81392 15 days ago |
0-13 13 seconds |
| 31738 |
robertmaxton42 author:robertmaxton42 |
feat: quivers can be represented as functors from the walking quiver |
Add definitions and associated lemmas for representing quivers as functors from the category `1 ⇉ 0`, i.e. `WalkingParallelPairᵒᵖ`.
New definitions:
* `asFunctor` itself, which is defined as a bare function with an associated `Functorial` instance so that it can be used with generalized projection notation
* `src` and `tgt`, abbreviations for `F.map left.op` and `F.map right.op` for a functor `F : WalkingParallelPairᵒᵖ ⥤ Type w`
* `Vertex`, `Edges`, and `Edge`, abbreviations for `F.obj 0` (interpreted as the type of vertices), `F.obj 1` (interpreted as the total type of all edges), and `{e : F.obj 1 // src e = s ∧ tgt e = t}` for some pair of vertices `s` and `t` (interpreted as the hom-type `s ⟶ t`)
* `edgeOfEq`, the equivalent of `Quiver.homOfEq` for edges in quivers in functor form.
---
This PR begins the first of a series proving that the category `Quiv.{v, u}` is equivalent to the subcategory of $$\mathbf{PSh}(\mathbf{WQuiv}^\mathrm{op})$$ which are appropriately '`u`-small' and 'locally `v`-small'. The original PR (prior to the move to forks) created a custom type `WalkingQuiver` for this purpose; ultimately I found that `WalkingParallelPairᵒᵖ` served my purposes well enough.
Following this PR will be one constructing the adjoint `ofFunctor`, plus several showing that `asFunctor` and `ofFunctor` can be assembled into an equivalence and proving various properties of quivers in functor form necessary for the construction of colimits.
[](https://gitpod.io/from-referrer/)
|
t-category-theory
merge-conflict
awaiting-author
|
397/0 |
Mathlib.lean,Mathlib/CategoryTheory/Category/Quiv/AsOfFunctor.lean |
2 |
13 |
['github-actions', 'joelriou', 'mathlib4-merge-conflict-bot', 'robertmaxton42'] |
nobody |
15-81352 15 days ago |
15-81353 15 days ago |
0-1741 29 minutes |
| 30083 |
grunweg author:grunweg |
feat: local frames in a vector bundle |
We construct local frames on a vector from local trivialisations. The former constructs, given a trivialisation `e` of the vector bundle and a basis of the model fibre, `Basis.localFrame` is a local frame on `e.baseSet`
A future PR will use this to define the local extension of a tangent vector to a vector field near a point.
From the path towards geodesics and the Levi-Civita connection.
Co-authored-by: Patrick Massot [patrickmassot@free.fr](mailto:patrickmassot@free.fr)
---
- [x] depends on: #27021
- [x] depends on: #30338
- [x] depends on: #31542
- [ ] depends on: #31788
[](https://gitpod.io/from-referrer/)
|
t-differential-geometry
merge-conflict
awaiting-author
|
326/22 |
Mathlib/Algebra/Module/Equiv/Basic.lean,Mathlib/Geometry/Manifold/VectorBundle/LocalFrame.lean |
2 |
51 |
['github-actions', 'grunweg', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'ocfnash'] |
ocfnash assignee:ocfnash |
15-71343 15 days ago |
15-71345 15 days ago |
19-1569 19 days |
| 31587 |
JovanGerb author:JovanGerb |
Lean pr testing 11156 |
Testing the performance improvement given by not deleting cache so often when modifying the environment.
cf. https://github.com/leanprover/lean4/pull/11156
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict
WIP
|
760/625 |
Archive/Imo/Imo1988Q6.lean,Archive/Imo/Imo1997Q3.lean,Archive/Imo/Imo2024Q5.lean,Archive/MiuLanguage/Basic.lean,Archive/Wiedijk100Theorems/BallotProblem.lean,Cache/Requests.lean,Counterexamples/PolynomialIsDomain.lean,Mathlib.lean,Mathlib/Algebra/Algebra/NonUnitalSubalgebra.lean,Mathlib/Algebra/Algebra/Subalgebra/Basic.lean,Mathlib/Algebra/Algebra/Subalgebra/Lattice.lean,Mathlib/Algebra/BigOperators/Fin.lean,Mathlib/Algebra/BigOperators/Ring/Finset.lean,Mathlib/Algebra/Category/Ring/Constructions.lean,Mathlib/Algebra/CharP/Subring.lean,Mathlib/Algebra/ContinuedFractions/Computation/Approximations.lean,Mathlib/Algebra/ContinuedFractions/ConvergentsEquiv.lean,Mathlib/Algebra/DirectSum/Internal.lean,Mathlib/Algebra/Group/Fin/Basic.lean,Mathlib/Algebra/Group/Int/Even.lean,Mathlib/Algebra/Group/Submonoid/Membership.lean,Mathlib/Algebra/Group/Submonoid/Operations.lean,Mathlib/Algebra/Group/Subsemigroup/Operations.lean,Mathlib/Algebra/Homology/Augment.lean,Mathlib/Algebra/Homology/Embedding/Connect.lean,Mathlib/Algebra/Lie/LieTheorem.lean,Mathlib/Algebra/Lie/Nilpotent.lean,Mathlib/Algebra/Lie/Weights/Chain.lean,Mathlib/Algebra/Lie/Weights/RootSystem.lean,Mathlib/Algebra/Module/Submodule/Map.lean,Mathlib/Algebra/Module/ZLattice/Basic.lean,Mathlib/Algebra/Order/Archimedean/Basic.lean,Mathlib/Algebra/Order/CauSeq/Basic.lean,Mathlib/Algebra/Order/Field/Power.lean,Mathlib/Algebra/Order/Group/Unbundled/Int.lean,Mathlib/Algebra/Order/Module/HahnEmbedding.lean,Mathlib/Algebra/Order/Ring/Unbundled/Rat.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/Div.lean,Mathlib/Algebra/Polynomial/Factors.lean,Mathlib/Algebra/Polynomial/Homogenize.lean,Mathlib/Algebra/Polynomial/Laurent.lean,Mathlib/Algebra/Polynomial/RingDivision.lean,Mathlib/Algebra/Polynomial/SumIteratedDerivative.lean,Mathlib/Algebra/Ring/Action/Invariant.lean,Mathlib/Algebra/Ring/Ext.lean,Mathlib/Algebra/Ring/Periodic.lean,Mathlib/Algebra/Ring/Subsemiring/Defs.lean,Mathlib/Algebra/Star/Module.lean,Mathlib/Algebra/Star/NonUnitalSubalgebra.lean,Mathlib/Algebra/Star/Subalgebra.lean,Mathlib/AlgebraicGeometry/Modules/Tilde.lean,Mathlib/AlgebraicGeometry/SpreadingOut.lean,Mathlib/AlgebraicGeometry/StructureSheaf.lean,Mathlib/AlgebraicTopology/DoldKan/Degeneracies.lean,Mathlib/AlgebraicTopology/DoldKan/Faces.lean,Mathlib/AlgebraicTopology/Quasicategory/Basic.lean,Mathlib/AlgebraicTopology/SimplexCategory/Basic.lean,Mathlib/AlgebraicTopology/SimplicialSet/Horn.lean,Mathlib/Analysis/Asymptotics/Theta.lean,Mathlib/Analysis/Calculus/ContDiff/FaaDiBruno.lean,Mathlib/Analysis/Complex/UpperHalfPlane/Basic.lean,Mathlib/Analysis/Convex/Between.lean,Mathlib/Analysis/Convex/SpecificFunctions/Deriv.lean,Mathlib/Analysis/Convex/StdSimplex.lean,Mathlib/Analysis/Distribution/TemperateGrowth.lean,Mathlib/Analysis/InnerProductSpace/Projection/Basic.lean,Mathlib/Analysis/Matrix/Spectrum.lean,Mathlib/Analysis/Meromorphic/Basic.lean,Mathlib/Analysis/Normed/Affine/Simplex.lean,Mathlib/Analysis/Normed/Field/UnitBall.lean,Mathlib/Analysis/Normed/Group/SemiNormedGrp/Kernels.lean,Mathlib/Analysis/Normed/Module/Ball/RadialEquiv.lean,Mathlib/Analysis/Normed/Ring/Ultra.lean,Mathlib/Analysis/NormedSpace/MStructure.lean,Mathlib/Analysis/SpecialFunctions/Gamma/Beta.lean,Mathlib/Analysis/SpecialFunctions/Log/Basic.lean,Mathlib/Analysis/SpecialFunctions/Pow/NNReal.lean,Mathlib/Analysis/SpecialFunctions/Pow/Real.lean,Mathlib/CategoryTheory/ConcreteCategory/UnbundledHom.lean,Mathlib/CategoryTheory/Groupoid/Subgroupoid.lean,Mathlib/Combinatorics/Additive/AP/Three/Defs.lean,Mathlib/Combinatorics/Additive/FreimanHom.lean,Mathlib/Combinatorics/Quiver/Arborescence.lean,Mathlib/Combinatorics/Schnirelmann.lean,Mathlib/Combinatorics/SimpleGraph/Extremal/Turan.lean,Mathlib/Combinatorics/SimpleGraph/FiveWheelLike.lean,Mathlib/Combinatorics/SimpleGraph/Hamiltonian.lean,Mathlib/Combinatorics/SimpleGraph/Trails.lean,Mathlib/Computability/Primrec.lean,Mathlib/Control/Random.lean,Mathlib/Data/Char.lean,Mathlib/Data/ENNReal/Basic.lean,Mathlib/Data/ENNReal/Inv.lean,Mathlib/Data/FP/Basic.lean,Mathlib/Data/Fin/Basic.lean,Mathlib/Data/Fin/SuccPred.lean |
297 |
5 |
['JovanGerb', 'github-actions', 'leanprover-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
15-61303 15 days ago |
21-73622 21 days ago* |
21-73599 21 days* |
| 21269 |
658060 author:658060 |
feat(CategoryTheory/Topos): basic definitions and results in topos theory |
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 |
['658060', 'gio256', 'github-actions', 'joelriou', 'mathlib4-dependent-issues-bot'] |
nobody |
15-60275 15 days ago |
283-31243 9 months ago |
0-13879 3 hours |
| 22805 |
ScottCarnahan author:ScottCarnahan |
feat(FieldTheory/Finite): fixed points of Frobenius automorphism |
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 |
15-60263 15 days ago |
264-66121 8 months ago |
0-0 0 seconds |
| 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 |
15-60158 15 days ago |
149-22161 4 months ago |
8-28043 8 days |
| 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
merge-conflict
WIP
|
141/0 |
Mathlib.lean,Mathlib/Data/Prod/RevLex.lean |
2 |
5 |
['ScottCarnahan', 'YaelDillies', 'github-actions', 'mathlib4-merge-conflict-bot'] |
YaelDillies assignee:YaelDillies |
15-60144 15 days ago |
16-1890 16 days ago |
19-33859 19 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 |
15-60138 15 days ago |
86-41470 2 months ago |
31-47622 31 days |
| 25726 |
tb65536 author:tb65536 |
feat: 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 |
15-60110 15 days ago |
123-81301 4 months ago |
0-1 1 second |
| 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
merge-conflict
WIP
|
132/0 |
Mathlib.lean,Mathlib/RingTheory/HahnSeries/Addition.lean,Mathlib/RingTheory/HahnSeries/Binomial.lean,Mathlib/RingTheory/HahnSeries/HEval.lean,Mathlib/RingTheory/HahnSeries/Multiplication.lean |
5 |
14 |
['ScottCarnahan', 'github-actions', 'kbuzzard', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
kbuzzard assignee:kbuzzard |
15-60103 15 days ago |
16-1729 16 days ago |
80-45817 80 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
merge-conflict
awaiting-author
|
358/0 |
Mathlib.lean,Mathlib/MeasureTheory/VectorMeasure/Variation/Defs.lean |
2 |
33 |
['EtienneC30', 'github-actions', 'mathlib4-merge-conflict-bot', 'yoh-tanimoto'] |
EtienneC30 assignee:EtienneC30 |
15-60007 15 days ago |
16-1564 16 days ago |
42-9361 42 days |
| 26455 |
ScottCarnahan author:ScottCarnahan |
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
merge-conflict
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 |
8 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-merge-conflict-bot'] |
nobody |
15-59977 15 days ago |
16-1516 16 days ago |
0-17731 4 hours |
| 26770 |
Jun2M author:Jun2M |
feat(Combinatorics/Graph): subgraph relations 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
merge-conflict
|
375/1 |
Mathlib.lean,Mathlib/Combinatorics/Graph/Basic.lean,Mathlib/Combinatorics/Graph/Subgraph.lean |
3 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
awainverse assignee:awainverse |
15-59952 15 days ago |
16-1382 16 days ago |
137-36187 137 days |
| 26804 |
kckennylau author:kckennylau |
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 |
15-59930 15 days ago |
134-2181 4 months ago |
0-163 2 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`.
---
- [x] depends on: #26824
[](https://gitpod.io/from-referrer/)
|
t-category-theory
merge-conflict
|
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-59918 15 days ago |
unknown |
unknown |
| 26348 |
mans0954 author:mans0954 |
feat(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
merge-conflict
WIP
|
125/0 |
Mathlib.lean,Mathlib/Analysis/LocallyConvex/Prime.lean |
2 |
3 |
['github-actions', 'mans0954', 'mathlib4-merge-conflict-bot'] |
nobody |
15-59911 15 days ago |
28-41848 28 days ago |
5-43062 5 days |
| 26310 |
kckennylau author:kckennylau |
feat: binary forms |
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
merge-conflict
awaiting-author
label:t-algebra$ |
73/0 |
Mathlib.lean,Mathlib/RingTheory/MvPolynomial/BinaryForm.lean |
2 |
14 |
['MichaelStollBayreuth', 'github-actions', 'kckennylau', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'ocfnash'] |
ocfnash assignee:ocfnash |
15-59896 15 days ago |
16-1534 16 days ago |
57-1104 57 days |
| 26283 |
kckennylau author:kckennylau |
feat: resultant of polynomials |
---
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
merge-conflict
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 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
15-59872 15 days ago |
16-1543 16 days ago |
0-19 19 seconds |
| 28215 |
5hv5hvnk author:5hv5hvnk |
feat: 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
merge-conflict
awaiting-author
WIP
|
1266/0 |
Mathlib.lean,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 |
6 |
4 |
['github-actions', 'grunweg', 'mathlib4-merge-conflict-bot'] |
nobody |
15-59820 15 days ago |
15-59820 15 days ago |
12-41939 12 days |
| 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 |
15-59798 15 days ago |
99-49770 3 months ago |
0-78027 21 hours |
| 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
merge-conflict
awaiting-author
label:t-algebra$ |
66/0 |
Mathlib.lean,Mathlib/Algebra/Algebra/ReducedNorm.lean |
2 |
19 |
['Whysoserioushah', 'chrisflav', 'erdOne', 'eric-wieser', 'github-actions', 'kbuzzard', 'mathlib4-merge-conflict-bot'] |
chrisflav assignee:chrisflav |
15-59768 15 days ago |
16-902 16 days ago |
41-8846 41 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
merge-conflict
awaiting-author
label:t-algebra$ |
270/0 |
Mathlib.lean,Mathlib/RepresentationTheory/CrossProductAlgebra/Defs.lean,docs/references.bib |
3 |
9 |
['Whysoserioushah', 'YaelDillies', 'eric-wieser', 'github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
15-59757 15 days ago |
16-893 16 days ago |
5-63264 5 days |
| 29281 |
plp127 author:plp127 |
doc: `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
merge-conflict
|
2/3 |
Mathlib/Data/Fin/Embedding.lean |
1 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
15-59728 15 days ago |
74-69627 2 months ago |
18-38918 18 days |
| 29514 |
grunweg author:grunweg |
feat(CI): use more strict mode |
---
[](https://gitpod.io/from-referrer/)
|
CI
merge-conflict
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 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
15-59716 15 days ago |
40-68559 1 month ago |
0-1 1 second |
| 29574 |
JarodAlper author:JarodAlper |
feat: 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
merge-conflict
|
910/3 |
Mathlib.lean,Mathlib/RingTheory/LocalRing/EmbeddingDimension.lean,Mathlib/RingTheory/LocalRing/LocalRingDimension.lean,Mathlib/RingTheory/LocalRing/RegularLocalRings.lean,Mathlib/RingTheory/LocalRing/RingHom/Basic.lean,lake-manifest.json |
6 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
15-59709 15 days ago |
81-17039 2 months ago |
3-7974 3 days |
| 29788 |
robertmaxton42 author:robertmaxton42 |
feat(Topology): adds bundled continuous maps for sum, sigma, subtype, mapsto, inclusion |
Adds a collection of bundled continuous maps and homeomorphisms, and helper lemmas for working with their compositions.
Bundling of existing continuity lemmas:
* `ContinuousMap.subtypeVal`
* `ContinuousMap.inl` and `.inr`; `ContinuousMap.sum` bundles `Continuous.sumElim`; `ContinuousMap.sumMap`, which is a quotient map when both components are quotient maps
* `ContinuousMap.sigmaMap`, which is a quotient map when given a family of quotient maps
* `ContinuousMap.mapsTo` bundles `ContinuousOn.restrict_mapsTo`
New functions:
* `ContinuousMap.preimageValIncl : C(s ↓∩ t, t)` and `.inclPreimageVal C(s, t ↓∩ s)`, and their unbundled functions in `Set`
* `Homeomorph.Set.preimageVal` witnesses that the two are opposite directions of a homeomorphism
* Descending from a coherent set of subspaces is a quotient map
The primary use for these bundled maps is easy composition and the ability to introduce them by rewriting right-to-left: it is much more convenient to write `subtypeVal.comp _` than to use either the anonymous constructor (which doesn't work in any position without an expected type) or `ContinuousMap.mk` (which will disappear as soon as it is coerced to a function, making it difficult to use in mixed-categorical contexts where many maps can only be reduced by introducing a composition with some other map.)
This PR is part of a family of PRs that ultimately construct transformations in both directions between the concrete `Topology.RelCWComplex` and abstract `TopCat.RelativeCWComplex`. `.mapsTo` in particular bundles together a couple of potentially nontrivial proofs in a way that makes them easy to refer to later; I use it and `.subtypeVal` particularly heavily later in a dependent PR to build the cell inclusion maps on both sides of the equivalence.
---
[](https://gitpod.io/from-referrer/)
|
large-import
merge-conflict
|
226/3 |
Mathlib/Data/Set/Subset.lean,Mathlib/Topology/Category/TopCat/Limits/Products.lean,Mathlib/Topology/Coherent.lean,Mathlib/Topology/Constructions.lean,Mathlib/Topology/Constructions/SumProd.lean,Mathlib/Topology/ContinuousMap/Basic.lean,scripts/noshake.json |
7 |
15 |
['adamtopaz', 'github-actions', 'mathlib4-merge-conflict-bot', 'robertmaxton42'] |
adamtopaz assignee:adamtopaz |
15-59631 15 days ago |
18-62514 18 days ago |
58-43534 58 days |
| 30366 |
sinhp author:sinhp |
feat(CategoryTheory): The Preliminaries for Locally Cartesian Closed Categories |
See https://github.com/leanprover-community/mathlib4/pull/21525
This PR defines the basic preliminaries for defining locally cartesian closed categories (LCCCs).
First, we develop a computable implementation of pullbacks, by introducing a new type-class `ChosenPullback`. The non-computable `HasPullbacksAlong` and `HasPullbacks` predicates yield instances of `ChosenPullback` using global choice, but interestingly in the category of types every morphism has chosen pullbacks. Also, cartesian monoidal categories, morphisms to the terminal object and the product projections have chosen pullbacks. We prove that `ChosenPullback` has good closure properties, e.g., isos have chosen pullbacks, and composition of morphisms with chosen pullbacks have chosen pullbacks.
Separately, we prove that pull-push along a morphism with chosen pullbacks gives the (cartesian) binary product of that morphism, seen as an object of a slice category, and any other object of the same slice category. In fact, we also prove the stronger statement, namely that the pull-push composition `(Over.ChosenPullback.pullback Z.hom) ⋙ (Over.map Z.hom)` is naturally isomorphic to the right tensor product functor `_ × Y` in `Over X`. _This is going to be crucial in our mate-based approach to LCCCs_.
Also, using the calculus of mates we define certain natural isomorphisms involving `Over.star` and `Over.pullback` which will be used in defining the right adjoint to the pullback functor in the development of LCCCs.
---
[](https://gitpod.io/from-referrer/)
|
t-category-theory
merge-conflict
awaiting-author
|
4865/526 |
.github/build.in.yml,.github/workflows/bors.yml,.github/workflows/build.yml,.github/workflows/build_fork.yml,Mathlib.lean,Mathlib/Algebra/Algebra/Spectrum/Quasispectrum.lean,Mathlib/Algebra/BigOperators/Group/List/Defs.lean,Mathlib/Algebra/BrauerGroup/Defs.lean,Mathlib/Algebra/Category/Grp/Subobject.lean,Mathlib/Algebra/Category/ModuleCat/Basic.lean,Mathlib/Algebra/Category/ModuleCat/Monoidal/Basic.lean,Mathlib/Algebra/Category/ModuleCat/Monoidal/Symmetric.lean,Mathlib/Algebra/Category/ModuleCat/Semi.lean,Mathlib/Algebra/CharP/Frobenius.lean,Mathlib/Algebra/Colimit/Ring.lean,Mathlib/Algebra/Field/MinimalAxioms.lean,Mathlib/Algebra/GroupWithZero/Hom.lean,Mathlib/Algebra/Homology/ComplexShapeSigns.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/Basic.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/Linear.lean,Mathlib/Algebra/Homology/DerivedCategory/Linear.lean,Mathlib/Algebra/Homology/HomologySequenceLemmas.lean,Mathlib/Algebra/Homology/HomotopyCategory/HomologicalFunctor.lean,Mathlib/Algebra/Homology/HomotopyCategory/ShiftSequence.lean,Mathlib/Algebra/Lie/CartanExists.lean,Mathlib/AlgebraicGeometry/Modules/Presheaf.lean,Mathlib/AlgebraicTopology/SimplexCategory/Defs.lean,Mathlib/AlgebraicTopology/SimplicialSet/AnodyneExtensions/IsUniquelyCodimOneFace.lean,Mathlib/AlgebraicTopology/SimplicialSet/AnodyneExtensions/Pairing.lean,Mathlib/AlgebraicTopology/SimplicialSet/Monoidal.lean,Mathlib/AlgebraicTopology/SimplicialSet/Nerve.lean,Mathlib/AlgebraicTopology/SimplicialSet/NerveAdjunction.lean,Mathlib/AlgebraicTopology/SimplicialSet/NonDegenerateSimplicesSubcomplex.lean,Mathlib/AlgebraicTopology/SimplicialSet/StdSimplex.lean,Mathlib/Analysis/Analytic/ChangeOrigin.lean,Mathlib/Analysis/Calculus/FDeriv/Prod.lean,Mathlib/Analysis/Calculus/IteratedDeriv/ConvergenceOnBall.lean,Mathlib/Analysis/Complex/OperatorNorm.lean,Mathlib/Analysis/Distribution/ContDiffMapSupportedIn.lean,Mathlib/Analysis/Distribution/SchwartzSpace.lean,Mathlib/Analysis/Distribution/TemperateGrowth.lean,Mathlib/Analysis/Meromorphic/TrailingCoefficient.lean,Mathlib/Analysis/Normed/Ring/WithAbs.lean,Mathlib/Analysis/SpecialFunctions/Log/PosLog.lean,Mathlib/CategoryTheory/Abelian/GrothendieckAxioms/Basic.lean,Mathlib/CategoryTheory/Abelian/GrothendieckAxioms/Sheaf.lean,Mathlib/CategoryTheory/Adjunction/AdjointFunctorTheorems.lean,Mathlib/CategoryTheory/Adjunction/Basic.lean,Mathlib/CategoryTheory/Adjunction/CompositionIso.lean,Mathlib/CategoryTheory/Adjunction/Mates.lean,Mathlib/CategoryTheory/Bicategory/Strict/Pseudofunctor.lean,Mathlib/CategoryTheory/Category/ULift.lean,Mathlib/CategoryTheory/Closed/Cartesian.lean,Mathlib/CategoryTheory/Comma/StructuredArrow/Small.lean,Mathlib/CategoryTheory/ComposableArrows.lean,Mathlib/CategoryTheory/Discrete/StructuredArrow.lean,Mathlib/CategoryTheory/EssentiallySmall.lean,Mathlib/CategoryTheory/Filtered/Final.lean,Mathlib/CategoryTheory/Functor/KanExtension/Pointwise.lean,Mathlib/CategoryTheory/Generator/Abelian.lean,Mathlib/CategoryTheory/Generator/Basic.lean,Mathlib/CategoryTheory/Generator/StrongGenerator.lean,Mathlib/CategoryTheory/GuitartExact/KanExtension.lean,Mathlib/CategoryTheory/IsConnected.lean,Mathlib/CategoryTheory/Limits/Filtered.lean,Mathlib/CategoryTheory/Limits/Final.lean,Mathlib/CategoryTheory/Limits/Final/Connected.lean,Mathlib/CategoryTheory/Limits/Final/Type.lean,Mathlib/CategoryTheory/Limits/HasLimits.lean,Mathlib/CategoryTheory/Limits/Preserves/Basic.lean,Mathlib/CategoryTheory/Limits/Preserves/Filtered.lean,Mathlib/CategoryTheory/Limits/Shapes/BinaryProducts.lean,Mathlib/CategoryTheory/Limits/Types/ColimitType.lean,Mathlib/CategoryTheory/LocallyCartesianClosed/Prelim.lean,Mathlib/CategoryTheory/Monoidal/Cartesian/Basic.lean,Mathlib/CategoryTheory/ObjectProperty/ClosedUnderIsomorphisms.lean,Mathlib/CategoryTheory/ObjectProperty/CompleteLattice.lean,Mathlib/CategoryTheory/ObjectProperty/LimitsClosure.lean,Mathlib/CategoryTheory/ObjectProperty/LimitsOfShape.lean,Mathlib/CategoryTheory/ObjectProperty/Small.lean,Mathlib/CategoryTheory/Presentable/IsCardinalFiltered.lean,Mathlib/CategoryTheory/Shift/ShiftedHom.lean,Mathlib/CategoryTheory/Sites/Descent/IsPrestack.lean,Mathlib/CategoryTheory/Sites/Equivalence.lean,Mathlib/CategoryTheory/Sites/LeftExact.lean,Mathlib/CategoryTheory/Sites/PreservesSheafification.lean,Mathlib/CategoryTheory/Sites/Whiskering.lean,Mathlib/Combinatorics/Enumerative/Bell.lean,Mathlib/Condensed/Discrete/Basic.lean,Mathlib/Condensed/Light/AB.lean,Mathlib/Condensed/Light/CartesianClosed.lean,Mathlib/Condensed/Light/Instances.lean,Mathlib/Condensed/Light/Module.lean,Mathlib/Data/Rel/Separated.lean,Mathlib/FieldTheory/PerfectClosure.lean,Mathlib/Geometry/Manifold/IsManifold/ExtChartAt.lean,Mathlib/Geometry/Manifold/MFDeriv/SpecificFunctions.lean,Mathlib/GroupTheory/ArchimedeanDensely.lean,Mathlib/GroupTheory/OrderOfElement.lean,Mathlib/GroupTheory/SpecificGroups/Cyclic.lean |
131 |
40 |
['github-actions', 'joelriou', 'mathlib4-merge-conflict-bot', 'sinhp'] |
nobody |
15-59595 15 days ago |
23-52543 23 days ago |
4-48785 4 days |
| 30855 |
Ruben-VandeVelde author:Ruben-VandeVelde |
fix: deprecate IsTotal in favour of Std.Total |
---
[](https://gitpod.io/from-referrer/)
|
RFC
merge-conflict
|
208/111 |
Mathlib/Algebra/Group/Basic.lean,Mathlib/Algebra/Order/Archimedean/Class.lean,Mathlib/Algebra/Order/GroupWithZero/Canonical.lean,Mathlib/Algebra/Order/Ring/Canonical.lean,Mathlib/Data/Finset/Sort.lean,Mathlib/Data/List/Sort.lean,Mathlib/Data/Multiset/Sort.lean,Mathlib/Data/Nat/PartENat.lean,Mathlib/Data/Ordmap/Invariants.lean,Mathlib/Data/Ordmap/Ordset.lean,Mathlib/Data/Prod/Basic.lean,Mathlib/Data/Prod/Lex.lean,Mathlib/Data/Real/Basic.lean,Mathlib/Data/Sigma/Lex.lean,Mathlib/Data/Sigma/Order.lean,Mathlib/Data/Sum/Order.lean,Mathlib/Logic/Encodable/Basic.lean,Mathlib/Order/Antisymmetrization.lean,Mathlib/Order/Basic.lean,Mathlib/Order/Comparable.lean,Mathlib/Order/Compare.lean,Mathlib/Order/Defs/Unbundled.lean,Mathlib/Order/Directed.lean,Mathlib/Order/Filter/FilterProduct.lean,Mathlib/Order/Lattice.lean,Mathlib/Order/PropInstances.lean,Mathlib/Order/RelClasses.lean,Mathlib/Order/RelIso/Basic.lean,Mathlib/Order/UpperLower/CompleteLattice.lean,Mathlib/Order/WithBot.lean,Mathlib/RingTheory/Valuation/ValuationRing.lean,Mathlib/RingTheory/Valuation/ValuationSubring.lean,Mathlib/Topology/EMetricSpace/BoundedVariation.lean |
33 |
3 |
['github-actions', 'linesthatinterlace', 'mathlib4-merge-conflict-bot'] |
alexjbest assignee:alexjbest |
14-28859 14 days ago |
16-70923 16 days ago |
24-78190 24 days |
| 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/)
|
awaiting-zulip
t-order
merge-conflict
|
175/181 |
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/GroupWithZero/Canonical.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/Computability/Reduce.lean,Mathlib/Data/DFinsupp/Order.lean,Mathlib/Data/Finset/Lattice/Basic.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/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/Preorder/Finsupp.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/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/Algebra/Module/ClosedSubmodule.lean,Mathlib/Topology/Category/TopCat/OpenNhds.lean,Mathlib/Topology/LocallyFinsupp.lean,Mathlib/Topology/MetricSpace/BundledFun.lean,Mathlib/Topology/UniformSpace/Basic.lean |
81 |
18 |
['JovanGerb', 'bryangingechen', 'eric-wieser', 'github-actions', 'j-loreaux', 'leanprover-bot', 'leanprover-community-bot-assistant', 'leanprover-community-mathlib4-bot', 'mathlib4-merge-conflict-bot'] |
Vierkantor assignee:Vierkantor |
13-60288 13 days ago |
13-60289 13 days ago |
24-8021 24 days |
| 31148 |
kex-y author:kex-y |
feat(Probability): Local and stable properties |
Defines local and stable properties which is useful for local martingales.
Co-authored-by: @RemyDegenne
---
[](https://gitpod.io/from-referrer/)
|
brownian
t-measure-probability
merge-conflict
WIP
|
644/0 |
Mathlib/Probability/Process/Filtration.lean,Mathlib/Probability/Process/LocalMonad.lean,Mathlib/Probability/Process/LocalProperty.lean,Mathlib/Probability/Process/Stopping.lean,Mathlib/Topology/Order/WithTop.lean |
5 |
4 |
['RemyDegenne', 'github-actions', 'kex-y', 'mathlib4-merge-conflict-bot'] |
nobody |
12-48098 12 days ago |
12-48098 12 days ago |
0-2992 49 minutes |
| 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
|
1974/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 |
11-74307 11 days ago |
84-74962 2 months ago |
0-0 0 seconds |
| 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* |
brownian
t-topology
merge-conflict
awaiting-author
|
453/1 |
Mathlib.lean,Mathlib/Data/Set/Accumulate.lean,Mathlib/Data/Set/Dissipate.lean,Mathlib/MeasureTheory/PiSystem.lean,Mathlib/Topology/Compactness/CompactSystem.lean |
5 |
27 |
['github-actions', 'mathlib4-merge-conflict-bot', 'pfaffelh', 'sgouezel'] |
PatrickMassot assignee:PatrickMassot |
11-65177 11 days ago |
11-65177 11 days ago |
70-65301 70 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* |
brownian
large-import
t-measure-probability
merge-conflict
awaiting-author
|
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 |
7 |
['github-actions', 'mathlib4-merge-conflict-bot', 'sgouezel'] |
kex-y assignee:kex-y |
11-65161 11 days ago |
11-65161 11 days ago |
31-59168 31 days |
| 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/)
- [x] depends on: #29988
- [x] depends on: #29989
- [x] depends on: #29990
- [x] depends on: #29991 |
t-algebra
merge-conflict
awaiting-author
label:t-algebra$ |
149/8 |
Mathlib.lean,Mathlib/Algebra/Group/Subgroup/Lattice.lean,Mathlib/RingTheory/RootsOfUnity/Basic.lean,Mathlib/RingTheory/RootsOfUnity/PrimitiveRoots.lean,Mathlib/RingTheory/Torsion.lean |
5 |
35 |
['chrisflav', 'github-actions', 'kckennylau', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'pechersky'] |
chrisflav assignee:chrisflav |
11-32774 11 days ago |
11-32901 11 days ago |
48-68722 48 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
|
971/371 |
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/Monoid/WithTop.lean,Mathlib/Algebra/Order/Ring/WithTop.lean,Mathlib/Algebra/Polynomial/Degree/Definitions.lean,Mathlib/Algebra/Polynomial/Degree/Operations.lean,Mathlib/Analysis/BoxIntegral/Box/Basic.lean,Mathlib/Analysis/BoxIntegral/Partition/Additive.lean,Mathlib/Analysis/BoxIntegral/Partition/Basic.lean,Mathlib/Analysis/BoxIntegral/Partition/Split.lean,Mathlib/Analysis/BoxIntegral/Partition/SubboxInduction.lean,Mathlib/Analysis/Meromorphic/Order.lean,Mathlib/Analysis/SpecialFunctions/Pow/NNReal.lean,Mathlib/Data/Countable/Basic.lean,Mathlib/Data/ENNReal/Basic.lean,Mathlib/Data/ENNReal/Operations.lean,Mathlib/Data/ENat/Defs.lean,Mathlib/Data/EReal/Operations.lean,Mathlib/Data/Finset/WithBot.lean,Mathlib/Data/Fintype/WithTopBot.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/Geometry/Manifold/PartitionOfUnity.lean,Mathlib/GroupTheory/ArchimedeanDensely.lean,Mathlib/Logic/Embedding/WithBot.lean,Mathlib/Logic/Equiv/WithBot.lean,Mathlib/MeasureTheory/Constructions/BorelSpace/Real.lean,Mathlib/MeasureTheory/Group/Measure.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/BooleanAlgebra.lean,Mathlib/Order/WithBot/NAry.lean,Mathlib/RingTheory/OrderOfVanishing.lean,Mathlib/RingTheory/UniqueFactorizationDomain/FactorSet.lean,Mathlib/SetTheory/Cardinal/ENat.lean,Mathlib/Topology/Algebra/Ring/Real.lean,Mathlib/Topology/Category/LightProfinite/Sequence.lean,Mathlib/Topology/Compactification/OnePoint/Basic.lean,Mathlib/Topology/Instances/ENat.lean,MathlibTest/lift.lean |
56 |
17 |
['eric-wieser', 'github-actions', 'kim-em', 'mathlib4-merge-conflict-bot'] |
nobody |
10-81014 10 days ago |
10-81015 10 days ago |
70-55654 70 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* |
merge-conflict
WIP
|
7956/304 |
Mathlib.lean,Mathlib/Algebra/Lie/Basic.lean,Mathlib/Algebra/Lie/ChevalleyEilenberg.lean,Mathlib/Algebra/Lie/Cochain.lean,Mathlib/Algebra/Lie/Cocycle.lean,Mathlib/Algebra/Lie/Extension.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 |
10-78091 10 days ago |
unknown |
unknown |
| 28933 |
artie2000 author:artie2000 |
chore(Data): correct definition for `single_apply` |
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict
WIP
|
42/40 |
Mathlib/Data/DFinsupp/Defs.lean,Mathlib/Data/DFinsupp/Sigma.lean,Mathlib/Data/Finsupp/Basic.lean,Mathlib/Data/Finsupp/Lex.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/DFinsupp.lean,Mathlib/LinearAlgebra/Finsupp/Defs.lean,Mathlib/LinearAlgebra/Finsupp/LinearCombination.lean,Mathlib/LinearAlgebra/Finsupp/Supported.lean,Mathlib/LinearAlgebra/Multilinear/DFinsupp.lean,Mathlib/LinearAlgebra/StdBasis.lean |
15 |
3 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
10-77282 10 days ago |
10-77283 10 days ago |
3-80673 3 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/)
- [x] depends on: #26829
|
t-topology
merge-conflict
awaiting-author
|
219/26 |
Mathlib.lean,Mathlib/NumberTheory/Padics/LinearTopology.lean,Mathlib/Topology/Algebra/Valued/LinearTopology.lean,Mathlib/Topology/Algebra/Valued/ValuationTopology.lean,Mathlib/Topology/Algebra/Valued/ValuedField.lean |
5 |
55 |
['ADedecker', 'erdOne', 'faenuccio', 'github-actions', 'jcommelin', 'leanprover-community-bot-assistant', 'loefflerd', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'pechersky'] |
jcommelin assignee:jcommelin |
10-72896 10 days ago |
10-72896 10 days ago |
36-12989 36 days |
| 26912 |
pechersky author:pechersky |
chore(Algebra/Ring/Subring): simp tag `Subring.smul_def` |
s-multiplying by a subtype is easiest to manipulate when both terms are in the ambient type. Many places that had to use the _def lemma for a rewrite, or to include it in a simp set, no longer have to.
Ported from #25308
---
[](https://gitpod.io/from-referrer/)
I found this being not-simp frustrating when talking about submodules over a valuation subring. |
t-algebra
merge-conflict
label:t-algebra$ |
67/66 |
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/WeylGroup.lean,Mathlib/RingTheory/Etale/Kaehler.lean,Mathlib/RingTheory/Ideal/Over.lean,Mathlib/RingTheory/LocalProperties/Projective.lean,Mathlib/RingTheory/Localization/InvSubmonoid.lean,Mathlib/RingTheory/OreLocalization/Basic.lean |
25 |
25 |
['artie2000', 'eric-wieser', 'github-actions', 'j-loreaux', 'kckennylau', 'leanprover-bot', 'leanprover-radar', 'linesthatinterlace', 'mathlib4-merge-conflict-bot', 'pechersky'] |
joelriou assignee:joelriou |
10-69017 10 days ago |
10-69018 10 days ago |
64-44898 64 days |
| 27756 |
grunweg author:grunweg |
feat: `Weak(Pseudo)EMetricSpace`, generalises `(Pseudo)EMetricSpace` |
---
[](https://gitpod.io/from-referrer/)
|
carleson
t-topology
merge-conflict
WIP
|
142/36 |
Mathlib/Topology/EMetricSpace/Defs.lean,Mathlib/Topology/Instances/ENNReal/Lemmas.lean |
2 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
10-57647 10 days ago |
10-57649 10 days ago |
0-2 2 seconds |
| 30904 |
vihdzp author:vihdzp |
chore: golf `Finsupp.single` lemmas |
In particular, we make the coercion `⇑(single a b) = Pi.single a b` a `simp` lemma.
---
- [ ] depends on: #30905
[](https://gitpod.io/from-referrer/)
|
t-data
merge-conflict
|
21/31 |
Mathlib/Data/Finsupp/Single.lean |
1 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
10-46941 10 days ago |
10-46942 10 days ago |
0-0 0 seconds |
| 31463 |
harahu author:harahu |
Tidy documentation code blocks |
This PR will not be published in its current form. It is intended to be broken up into a collection of smaller PRs.
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict |
185/53 |
Mathlib/Lean/Expr/Basic.lean,Mathlib/Tactic/Choose.lean,Mathlib/Tactic/DeriveTraversable.lean,Mathlib/Tactic/GCongr/Core.lean,Mathlib/Tactic/Linarith/Frontend.lean,Mathlib/Tactic/Linter/PPRoundtrip.lean,Mathlib/Tactic/MinImports.lean,Mathlib/Tactic/MkIffOfInductiveProp.lean,Mathlib/Tactic/MoveAdd.lean,Mathlib/Tactic/Relation/Rfl.lean,Mathlib/Tactic/Relation/Symm.lean,Mathlib/Tactic/Simps/Basic.lean,Mathlib/Topology/Algebra/InfiniteSum/Defs.lean,Mathlib/Util/SynthesizeUsing.lean,MathlibTest/DoubleUnderscore.lean,MathlibTest/FindSyntax.lean,MathlibTest/depRewrite.lean,MathlibTest/meta.lean,MathlibTest/notation3.lean,find_unmatched_backticks.py,unmatched_backticks_report.txt |
21 |
6 |
['github-actions', 'grunweg', 'harahu', 'mathlib4-merge-conflict-bot'] |
nobody |
10-46806 10 days ago |
10-46807 10 days ago |
0-0 0 seconds |
| 31595 |
astrainfinita author:astrainfinita |
chore: redefine `Ideal.IsPrime` |
Redefine `Ideal.IsPrime` to make it correct for non-commutative cases
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
awaiting-author
label:t-algebra$ |
209/101 |
Mathlib/Algebra/Order/Ring/Ordering/Defs.lean,Mathlib/AlgebraicGeometry/StructureSheaf.lean,Mathlib/RingTheory/DedekindDomain/Ideal/Lemmas.lean,Mathlib/RingTheory/GradedAlgebra/Radical.lean,Mathlib/RingTheory/Ideal/AssociatedPrime/Basic.lean,Mathlib/RingTheory/Ideal/IsPrimary.lean,Mathlib/RingTheory/Ideal/Maps.lean,Mathlib/RingTheory/Ideal/Maximal.lean,Mathlib/RingTheory/Ideal/Oka.lean,Mathlib/RingTheory/Ideal/Operations.lean,Mathlib/RingTheory/Ideal/Over.lean,Mathlib/RingTheory/Ideal/Pointwise.lean,Mathlib/RingTheory/Ideal/Prime.lean,Mathlib/RingTheory/Ideal/Prod.lean,Mathlib/RingTheory/Ideal/Quotient/Basic.lean,Mathlib/RingTheory/Localization/AtPrime/Basic.lean,Mathlib/RingTheory/Localization/Ideal.lean,Mathlib/RingTheory/Polynomial/Basic.lean,Mathlib/RingTheory/PrincipalIdealDomain.lean,Mathlib/RingTheory/Spectrum/Prime/Topology.lean,Mathlib/RingTheory/Valuation/Basic.lean |
21 |
13 |
['alreadydone', 'github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'mathlib4-merge-conflict-bot'] |
alreadydone assignee:alreadydone |
10-34934 10 days ago |
10-34935 10 days ago |
6-85888 6 days |
| 31948 |
ADedecker author:ADedecker |
feat: move `ContinuousSMul` to a finite extension with the module topology |
My motivation is the following: to define the topology on test functions (see #31806), we take the inductive limit in the category of *real* locally convex topological vector spaces (we don't want the result to depend on the base field!). But then, we need a way to get that complex-valued test functions are also a *complex* topological vector space, which we will obtain by combining this PR with [isModuleTopologyOfFiniteDimensional](https://leanprover-community.github.io/mathlib4_docs/Mathlib/Topology/Algebra/Module/FiniteDimension.html#isModuleTopologyOfFiniteDimensional).
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict |
109/57 |
Mathlib/Algebra/Algebra/Basic.lean,Mathlib/Algebra/Module/LinearMap/Basic.lean,Mathlib/Analysis/LocallyConvex/WeakDual.lean,Mathlib/FieldTheory/Fixed.lean,Mathlib/LinearAlgebra/LinearIndependent/Lemmas.lean,Mathlib/LinearAlgebra/Pi.lean,Mathlib/Topology/Algebra/Module/Basic.lean,Mathlib/Topology/Algebra/Module/ModuleTopology.lean |
8 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
10-31163 10 days ago |
10-31164 10 days ago |
0-0 0 seconds |
| 31972 |
harahu author:harahu |
chore: rewrite doc refs to file paths |
- replace doc/comment module references (Foo.Bar.Baz) with explicit file paths (Mathlib/Foo/Bar/Baz.lean) so links point to real files
- add scripts/replace_module_refs.py to automate the conversion for future cleanup (dry-run by default, --apply to rewrite)
- touch only docstrings/comments; no code changes
Co-authored by Codex.
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict |
738/527 |
Archive/Imo/Imo2019Q2.lean,Counterexamples/ZeroDivisorsInAddMonoidAlgebras.lean,Mathlib/Algebra/Algebra/Bilinear.lean,Mathlib/Algebra/BigOperators/Field.lean,Mathlib/Algebra/Category/ModuleCat/ChangeOfRings.lean,Mathlib/Algebra/Category/ModuleCat/LeftResolution.lean,Mathlib/Algebra/Category/ModuleCat/Monoidal/Basic.lean,Mathlib/Algebra/Category/ModuleCat/Products.lean,Mathlib/Algebra/Category/ModuleCat/Sheaf/Abelian.lean,Mathlib/Algebra/ContinuedFractions/Basic.lean,Mathlib/Algebra/ContinuedFractions/Computation/ApproximationCorollaries.lean,Mathlib/Algebra/ContinuedFractions/Computation/Approximations.lean,Mathlib/Algebra/ContinuedFractions/Computation/CorrectnessTerminating.lean,Mathlib/Algebra/ContinuedFractions/Translations.lean,Mathlib/Algebra/EuclideanDomain/Defs.lean,Mathlib/Algebra/GCDMonoid/Multiset.lean,Mathlib/Algebra/GradedMonoid.lean,Mathlib/Algebra/Group/Action/Defs.lean,Mathlib/Algebra/Group/Even.lean,Mathlib/Algebra/Group/Ext.lean,Mathlib/Algebra/Group/Pi/Basic.lean,Mathlib/Algebra/Group/Pi/Lemmas.lean,Mathlib/Algebra/Group/TypeTags/Basic.lean,Mathlib/Algebra/Group/ULift.lean,Mathlib/Algebra/GroupWithZero/Action/Basic.lean,Mathlib/Algebra/GroupWithZero/Action/Pi.lean,Mathlib/Algebra/GroupWithZero/Action/Prod.lean,Mathlib/Algebra/GroupWithZero/Action/Units.lean,Mathlib/Algebra/GroupWithZero/Basic.lean,Mathlib/Algebra/Homology/BifunctorAssociator.lean,Mathlib/Algebra/Homology/DerivedCategory/Basic.lean,Mathlib/Algebra/Homology/ExactSequence.lean,Mathlib/Algebra/Homology/LeftResolution/Reduced.lean,Mathlib/Algebra/Homology/Refinements.lean,Mathlib/Algebra/Homology/ShortComplex/RightHomology.lean,Mathlib/Algebra/Homology/ShortComplex/SnakeLemma.lean,Mathlib/Algebra/Homology/Square.lean,Mathlib/Algebra/ModEq.lean,Mathlib/Algebra/Module/Hom.lean,Mathlib/Algebra/Module/PID.lean,Mathlib/Algebra/Module/Submodule/Bilinear.lean,Mathlib/Algebra/Order/Hom/Basic.lean,Mathlib/Algebra/Order/Interval/Basic.lean,Mathlib/Algebra/Order/Monovary.lean,Mathlib/Algebra/Order/Ring/Unbundled/Basic.lean,Mathlib/Algebra/Order/Ring/Unbundled/Rat.lean,Mathlib/Algebra/Ring/SumsOfSquares.lean,Mathlib/Algebra/Squarefree/Basic.lean,Mathlib/Algebra/Star/Free.lean,Mathlib/AlgebraicGeometry/AffineScheme.lean,Mathlib/AlgebraicGeometry/AffineSpace.lean,Mathlib/AlgebraicGeometry/IdealSheaf/Subscheme.lean,Mathlib/AlgebraicGeometry/ResidueField.lean,Mathlib/AlgebraicGeometry/Sites/BigZariski.lean,Mathlib/AlgebraicGeometry/Sites/Pretopology.lean,Mathlib/AlgebraicTopology/FundamentalGroupoid/Basic.lean,Mathlib/AlgebraicTopology/Quasicategory/Nerve.lean,Mathlib/AlgebraicTopology/Quasicategory/StrictSegal.lean,Mathlib/AlgebraicTopology/SimplicialCategory/SimplicialObject.lean,Mathlib/AlgebraicTopology/TopologicalSimplex.lean,Mathlib/Analysis/Analytic/RadiusLiminf.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Integral.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/NonUnital.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Unital.lean,Mathlib/Analysis/CStarAlgebra/Matrix.lean,Mathlib/Analysis/CStarAlgebra/Module/Constructions.lean,Mathlib/Analysis/CStarAlgebra/Module/Defs.lean,Mathlib/Analysis/Calculus/Conformal/NormedSpace.lean,Mathlib/Analysis/Calculus/ContDiff/RestrictScalars.lean,Mathlib/Analysis/Calculus/FDeriv/Basic.lean,Mathlib/Analysis/Complex/Circle.lean,Mathlib/Analysis/Convex/Function.lean,Mathlib/Analysis/Convex/Jensen.lean,Mathlib/Analysis/Convex/SpecificFunctions/Deriv.lean,Mathlib/Analysis/Convex/SpecificFunctions/Pow.lean,Mathlib/Analysis/InnerProductSpace/Defs.lean,Mathlib/Analysis/InnerProductSpace/Laplacian.lean,Mathlib/Analysis/InnerProductSpace/LaxMilgram.lean,Mathlib/Analysis/InnerProductSpace/OfNorm.lean,Mathlib/Analysis/InnerProductSpace/Orthogonal.lean,Mathlib/Analysis/InnerProductSpace/l2Space.lean,Mathlib/Analysis/Meromorphic/IsolatedZeros.lean,Mathlib/Analysis/Normed/Algebra/Exponential.lean,Mathlib/Analysis/Normed/Group/Continuity.lean,Mathlib/Analysis/Normed/Group/FunctionSeries.lean,Mathlib/Analysis/Normed/Lp/PiLp.lean,Mathlib/Analysis/Normed/Lp/ProdLp.lean,Mathlib/Analysis/Normed/Module/WeakDual.lean,Mathlib/Analysis/Normed/Operator/BanachSteinhaus.lean,Mathlib/Analysis/Normed/Operator/BoundedLinearMaps.lean,Mathlib/Analysis/Normed/Operator/Completeness.lean,Mathlib/Analysis/Normed/Operator/Conformal.lean,Mathlib/Analysis/PSeriesComplex.lean,Mathlib/Analysis/SpecialFunctions/Complex/CircleAddChar.lean,Mathlib/Analysis/SpecialFunctions/Exponential.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Basic.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Complex.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Inverse.lean,Mathlib/CategoryTheory/Abelian/GrothendieckAxioms/Basic.lean,Mathlib/CategoryTheory/Abelian/Pseudoelements.lean |
367 |
5 |
['github-actions', 'grunweg', 'mathlib4-merge-conflict-bot'] |
nobody |
10-31161 10 days ago |
10-31163 10 days 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
merge-conflict
|
283/0 |
Mathlib.lean,Mathlib/Topology/UniformSpace/FineUniformity.lean,Mathlib/Topology/UniformSpace/Uniformizable.lean |
3 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
10-20285 10 days ago |
10-20286 10 days ago |
2-85349 2 days |
| 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
merge-conflict
awaiting-author
|
74/0 |
Mathlib/Combinatorics/SimpleGraph/Walk.lean |
1 |
19 |
['Rida-Hamadani', 'b-mehta', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
9-76948 9 days ago |
9-76949 9 days ago |
4-83551 4 days |
| 32095 |
grunweg author:grunweg |
chore: fix some explicitVarOfIff linter errors |
Needs a merge, and removing the linter changes... should be re-done and split out!
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict
please-adopt
WIP
|
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 |
0 |
[] |
nobody |
9-73929 9 days ago |
9-73929 9 days ago |
0-8 8 seconds |
| 26950 |
alreadydone author:alreadydone |
Primitives of holomorphic functions and path integral |
---
- [x] depends on: #22782
- [x] depends on: #24983
- [ ] depends on: #22771
[](https://gitpod.io/from-referrer/)
|
t-analysis
t-topology
merge-conflict
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 |
9-38200 9 days ago |
unknown |
unknown |
| 26884 |
alreadydone author:alreadydone |
Universal cover |
---
- [ ] depends on: #24983
- [ ] depends on: #22771
- [ ] depends on: #22782
[](https://gitpod.io/from-referrer/)
|
t-topology
merge-conflict
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 |
9-38190 9 days ago |
148-55712 4 months ago |
0-0 0 seconds |
| 29982 |
hrmacbeth author:hrmacbeth |
feat: new `isolate` tactic |
This PR adds a new tactic, `isolate`, which "solves for x" in an equation or relation. For example:
```lean
example (a b : ℝ) (f : ℝ → ℝ) : 5 * f a - 3 < b := by
isolate f a
-- new goal: `⊢ f a < (b + 3) / 5`
```
The `isolate` tactic may generate side goals, if these are necessary to justify the transformation. The tactic will attempt to justify such side goals using `positivity` (as in the above example), unification, or type class inference, but if unsuccessful will present them to the user. For example:
```lean
example (a b c : ℝ) (f : ℝ → ℝ) : c * f a - 3 < b := by
isolate f a
-- new goal: `⊢ f a < (b + 3) / c`
-- second (side) new goal: `⊢ 0 < c`
```
The `isolate` tactic is extensible. Coverage may be extended to new relations and new operations-to-be-undone by tagging appropriate lemmas with the new `@[isolate]` attribute.
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-meta
merge-conflict
awaiting-author
|
861/1 |
Mathlib.lean,Mathlib/Analysis/SpecialFunctions/Log/Basic.lean,Mathlib/Analysis/SpecialFunctions/Pow/Real.lean,Mathlib/Data/Real/Sqrt.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Isolate.lean,Mathlib/Tactic/Isolate/Core.lean,Mathlib/Tactic/Isolate/Tagging.lean,Mathlib/Tactic/Relation/Symm.lean,MathlibTest/Isolate/Heavyweight.lean,MathlibTest/Isolate/Lightweight.lean,scripts/noshake.json |
12 |
41 |
['JovanGerb', 'PatrickMassot', 'Vierkantor', 'github-actions', 'hrmacbeth', 'kim-em', 'mathlib4-merge-conflict-bot'] |
JovanGerb assignee:JovanGerb |
9-19532 9 days ago |
18-62512 18 days ago |
49-50475 49 days |
| 29899 |
eric-wieser author:eric-wieser |
chore: add `=Q` arguments to ring casting operations |
This also detects an `isDefeq` which is unifying across universes and types, which I remember rumors about being sometimes a bad idea.
I'm a little worried that the `=Q` design here runs into DTT hell, but it works in the one place that is "Qq-clean" right now, so I'd be inclined to apply it to help us learn more about the pattern in future.
---
[](https://gitpod.io/from-referrer/)
|
t-meta
merge-conflict
|
36/23 |
Mathlib/Tactic/Ring/Basic.lean |
1 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
9-14980 9 days ago |
9-14981 9 days ago |
0-0 0 seconds |
| 31007 |
kckennylau author:kckennylau |
feat(RingTheory): generalise perfection to monoids |
1. We generalise `PerfectRing` to monoids (without changing the name).
2. We move `Submonoid.perfection` and `Ring.Perfection` to the already existing `Perfection` namespace, which solves the problem that `Ring.Perfection` and its lemmas `Perfection.xxx` are in different namespaces. Also, the monoid perfection and right perfection have the same underlying set, so this unify the two approaches.
3. `Perfection.lift` is now generalised to monoids: `liftMonoidHom : (M →* N) ≃ (M →* Perfection N p)` where `M` is a perfect monoid.
---
This is in preparation for a future PR following #30989.
[](https://gitpod.io/from-referrer/)
|
merge-conflict |
251/127 |
Mathlib/FieldTheory/Perfect.lean,Mathlib/FieldTheory/PerfectClosure.lean,Mathlib/RingTheory/Perfection.lean,Mathlib/RingTheory/Perfectoid/Untilt.lean |
4 |
34 |
['github-actions', 'jjdishere', 'kckennylau', 'mathlib4-merge-conflict-bot', 'pechersky'] |
nobody |
9-11846 9 days ago |
9-11847 9 days ago |
21-19809 21 days |
| 31920 |
thorimur author:thorimur |
test: `env_linter` for unused decidable instances |
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict |
128/0 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter.lean,Mathlib/Tactic/Linter/DirectoryDependency.lean,Mathlib/Tactic/Linter/UnusedAssumptionInType.lean |
5 |
19 |
['github-actions', 'leanprover-bot', 'leanprover-radar', 'mathlib4-merge-conflict-bot', 'thorimur'] |
nobody |
9-11594 9 days ago |
9-11594 9 days ago |
0-0 0 seconds |
| 32066 |
thorimur author:thorimur |
bench: alternate implementation of unusedDecidable |
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict |
554/4 |
Mathlib.lean,Mathlib/Computability/Halting.lean,Mathlib/Data/Fintype/Quotient.lean,Mathlib/Lean/Elab/InfoTree.lean,Mathlib/Lean/Environment.lean,Mathlib/Lean/Expr/Basic.lean,Mathlib/Logic/Encodable/Basic.lean,Mathlib/RingTheory/TensorProduct/IsBaseChangeFree.lean,Mathlib/RingTheory/TensorProduct/IsBaseChangePi.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter.lean,Mathlib/Tactic/Linter/DirectoryDependency.lean,Mathlib/Tactic/Linter/UnusedInstancesInType.lean,MathlibTest/UnusedInstancesInType.lean |
14 |
6 |
['github-actions', 'leanprover-bot', 'leanprover-radar', 'mathlib4-merge-conflict-bot', 'thorimur'] |
nobody |
9-11205 9 days ago |
9-11207 9 days ago |
0-0 0 seconds |
| 30047 |
ooovi author:ooovi |
feat(Combinatorics/SimpleGraph): edge labellings |
Add edge labellings for `SimpleGraph` as well as some basic lemmata.
---
This is mostly a cleaned up part of @b-mehta's lean4 port of their [formalisation of an exponentially better upper bound on Ramsey numbers ](https://github.com/b-mehta/ExponentialRamsey/). I need these definitions for another project on Ramsey theory.
[](https://gitpod.io/from-referrer/)
|
maintainer-merge
t-combinatorics
merge-conflict
awaiting-author
|
234/3 |
Mathlib.lean,Mathlib/Combinatorics/SimpleGraph/Basic.lean,Mathlib/Combinatorics/SimpleGraph/EdgeLabelling.lean,Mathlib/Combinatorics/SimpleGraph/Regularity/Increment.lean,Mathlib/Combinatorics/SimpleGraph/Triangle/Counting.lean |
5 |
54 |
['YaelDillies', 'b-mehta', 'github-actions', 'mathlib4-merge-conflict-bot', 'ocfnash', 'ooovi', 'vlad902'] |
b-mehta assignee:b-mehta |
8-62345 8 days ago |
16-251 16 days ago |
34-69915 34 days |
| 26138 |
xroblot author:xroblot |
Development branch (2) |
---
|
merge-conflict
WIP
|
331/70 |
Mathlib/Algebra/Algebra/Subalgebra/Lattice.lean,Mathlib/FieldTheory/Finite/GaloisField.lean,Mathlib/FieldTheory/Galois/IsGaloisGroup.lean,Mathlib/FieldTheory/IntermediateField/Adjoin/Defs.lean,Mathlib/NumberTheory/NumberField/CMField.lean,Mathlib/NumberTheory/NumberField/Cyclotomic/Embeddings.lean,Mathlib/NumberTheory/NumberField/InfinitePlace/Basic.lean,Mathlib/NumberTheory/NumberField/InfinitePlace/Embeddings.lean,Mathlib/NumberTheory/NumberField/InfinitePlace/Ramification.lean,Mathlib/NumberTheory/NumberField/InfinitePlace/TotallyRealComplex.lean,Mathlib/Sandbox.lean |
11 |
n/a |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-merge-conflict-bot'] |
nobody |
8-56462 8 days 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
awaiting-author
|
53/48 |
Mathlib/Data/Nat/Prime/Defs.lean |
1 |
3 |
['digama0', 'github-actions', 'leanprover-community-bot-assistant'] |
nobody |
7-85174 7 days ago |
7-85174 7 days ago |
8-58125 8 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
merge-conflict
awaiting-author
|
44/22 |
Mathlib/Data/Int/GCD.lean |
1 |
6 |
['astrainfinita', 'b-mehta', 'eric-wieser', 'github-actions', 'mathlib4-merge-conflict-bot', 'nomeata', 'urkud'] |
nobody |
7-75704 7 days ago |
7-75705 7 days ago |
58-34020 58 days |
| 31152 |
FernandoChu author:FernandoChu |
feat(CategoryTheory): regular categories have strong-epi-mono factorisations |
This PR defines regular categories and shows that these have strong-epi-mono factorisations. A follow up PR will prove frobenius reciprocity.
- [x] depends on: https://github.com/leanprover-community/mathlib4/pull/31145
---
This is a prerequisite of the [MTT project](https://github.com/kyoDralliam/model-theory-topos), which aims to use the internal language of toposes to reason about e.g. sheaves. |
t-category-theory
merge-conflict
awaiting-author
|
223/0 |
Mathlib.lean,Mathlib/CategoryTheory/Limits/Shapes/KernelPair.lean,Mathlib/CategoryTheory/Limits/Shapes/RegularMono.lean,Mathlib/CategoryTheory/RegularCategory/Basic.lean,docs/references.bib |
5 |
22 |
['FernandoChu', 'dagurtomas', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
dagurtomas assignee:dagurtomas |
7-59636 7 days ago |
7-59636 7 days ago |
7-8323 7 days |
| 31361 |
alreadydone author:alreadydone |
feat(Algebra/Order): convex subgroups |
---
[](https://gitpod.io/from-referrer/)
|
t-order
t-algebra
merge-conflict
awaiting-author
label:t-algebra$ |
379/0 |
Mathlib.lean,Mathlib/Algebra/Order/Archimedean/Class.lean,Mathlib/Algebra/Order/Group/Convex.lean,Mathlib/Order/Birkhoff.lean |
4 |
11 |
['alreadydone', 'github-actions', 'kckennylau', 'mathlib4-merge-conflict-bot', 'vihdzp', 'wwylele'] |
Vierkantor assignee:Vierkantor |
6-54298 6 days ago |
6-76963 6 days ago |
11-66060 11 days |
| 32143 |
edegeltje author:edegeltje |
test: Add an abbrev for `Cat.Hom2.toNatTrans.app` |
This PR is built upon #31807, to trigger CI into building this test and see where fixes are needed
---
[](https://gitpod.io/from-referrer/)
|
t-category-theory
merge-conflict
awaiting-author
WIP
|
820/606 |
Mathlib/Algebra/Category/ModuleCat/Pseudofunctor.lean,Mathlib/AlgebraicTopology/Quasicategory/StrictBicategory.lean,Mathlib/AlgebraicTopology/SimplicialSet/HomotopyCat.lean,Mathlib/AlgebraicTopology/SimplicialSet/Nerve.lean,Mathlib/AlgebraicTopology/SimplicialSet/NerveAdjunction.lean,Mathlib/CategoryTheory/Bicategory/CatEnriched.lean,Mathlib/CategoryTheory/Bicategory/Functor/Cat.lean,Mathlib/CategoryTheory/Bicategory/Grothendieck.lean,Mathlib/CategoryTheory/Category/Cat.lean,Mathlib/CategoryTheory/Category/Cat/Adjunction.lean,Mathlib/CategoryTheory/Category/Cat/AsSmall.lean,Mathlib/CategoryTheory/Category/Cat/CartesianClosed.lean,Mathlib/CategoryTheory/Category/Cat/Limit.lean,Mathlib/CategoryTheory/Category/Cat/Op.lean,Mathlib/CategoryTheory/Category/Cat/Terminal.lean,Mathlib/CategoryTheory/Category/Grpd.lean,Mathlib/CategoryTheory/Category/Quiv.lean,Mathlib/CategoryTheory/Category/ReflQuiv.lean,Mathlib/CategoryTheory/CodiscreteCategory.lean,Mathlib/CategoryTheory/Comma/Over/Basic.lean,Mathlib/CategoryTheory/Comma/StructuredArrow/Final.lean,Mathlib/CategoryTheory/Comma/StructuredArrow/Functor.lean,Mathlib/CategoryTheory/Elements.lean,Mathlib/CategoryTheory/FiberedCategory/Grothendieck.lean,Mathlib/CategoryTheory/Filtered/Grothendieck.lean,Mathlib/CategoryTheory/Functor/KanExtension/Adjunction.lean,Mathlib/CategoryTheory/Grothendieck.lean,Mathlib/CategoryTheory/Groupoid/FreeGroupoidOfCategory.lean,Mathlib/CategoryTheory/IsomorphismClasses.lean,Mathlib/CategoryTheory/Join/Pseudofunctor.lean,Mathlib/CategoryTheory/Limits/Final.lean,Mathlib/CategoryTheory/Limits/Shapes/Grothendieck.lean,Mathlib/CategoryTheory/Monoidal/Cartesian/Cat.lean,Mathlib/CategoryTheory/SingleObj.lean,Mathlib/CategoryTheory/Sites/Descent/DescentData.lean,Mathlib/CategoryTheory/Sites/Descent/IsPrestack.lean,Mathlib/CategoryTheory/Sites/PseudofunctorSheafOver.lean,Mathlib/CategoryTheory/WithTerminal/Basic.lean,Mathlib/Order/Category/Preord.lean,Mathlib/Tactic/CategoryTheory/ToApp.lean,MathlibTest/CategoryTheory/ToApp.lean |
41 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
6-52969 6 days ago |
6-52969 6 days ago |
0-0 0 seconds |
| 29934 |
smmercuri author:smmercuri |
feat(Field/WithAbs): the lift of a ring homomorphism from `WithAbs v` to `WithAbs w` to their completions |
If `σ` is a compatible ring homomomorphism between `WithAbs v` and `WithAbs w` then this extends to a natural ring homomorphism between completions `v.Completion` and `w.Completion`.
Also fix some defeq abuse in `Field/WithAbs`.
---
- [ ] depends on: #29969
[](https://gitpod.io/from-referrer/)
|
FLT
merge-conflict
WIP
|
104/48 |
Mathlib/Analysis/Normed/Field/WithAbs.lean,Mathlib/NumberTheory/NumberField/AdeleRing.lean,Mathlib/NumberTheory/NumberField/InfinitePlace/Completion.lean,Mathlib/Topology/MetricSpace/Completion.lean |
4 |
4 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
6-49775 6 days ago |
6-49778 6 days ago |
0-2230 37 minutes |
| 29933 |
smmercuri author:smmercuri |
chore: fix `def` naming isses in `Normed/Field/WithAbs.lean` |
---
- [x] depends on: #29932
[](https://gitpod.io/from-referrer/)
|
merge-conflict
WIP
|
33/23 |
Mathlib/Analysis/Normed/Field/WithAbs.lean,Mathlib/NumberTheory/NumberField/AdeleRing.lean,Mathlib/NumberTheory/NumberField/InfinitePlace/Completion.lean |
3 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
6-49247 6 days ago |
6-49248 6 days ago |
1-17350 1 day |
| 31377 |
CoolRmal author:CoolRmal |
feat: a series of smooth functions that converges (locally) uniformly is smooth |
The main theorem is the proof that an infinite sum of $C^n$ functions on a one-dimensional domain which converges locally uniformly is $C^n$ and related results.
This should be compared with [contDiff_tsum](https://leanprover-community.github.io/mathlib4_docs/Mathlib/Analysis/Calculus/SmoothSeries.html#contDiff_tsum) where the same result is proved for functions on an arbitrary domain but with a slightly stronger convergence assumption.
The main motivation for this PR is the [#mathlib4 > Tychonov's Counterexample for the Heat Equation](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Tychonov's.20Counterexample.20for.20the.20Heat.20Equation/with/547367912).
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-topology
merge-conflict
awaiting-author
|
115/22 |
Mathlib/Analysis/Calculus/SmoothSeries.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Cotangent.lean,Mathlib/NumberTheory/ModularForms/EisensteinSeries/QExpansion.lean,Mathlib/Topology/Algebra/InfiniteSum/TsumUniformlyOn.lean,Mathlib/Topology/Algebra/InfiniteSum/UniformOn.lean |
5 |
19 |
['CoolRmal', 'github-actions', 'mathlib4-merge-conflict-bot', 'ocfnash', 'sgouezel'] |
ocfnash assignee:ocfnash |
6-48290 6 days ago |
6-48291 6 days ago |
8-15568 8 days |
| 30860 |
FormulaRabbit81 author:FormulaRabbit81 |
feat(Measure): prove the space of probability measures on a compact space is compact |
---
- [x] depends on: #30845
- [x] depends on: #28061
- [x] depends on #31656
- [x] depends on #31964
Note this lemma is currently in the wrong place and will be moved once completed
[](https://gitpod.io/from-referrer/) |
merge-conflict
WIP
|
248/34 |
Mathlib/Algebra/Order/Module/PositiveLinearMap.lean,Mathlib/MeasureTheory/Integral/RieszMarkovKakutani/NNReal.lean,Mathlib/MeasureTheory/Measure/FiniteMeasure.lean,Mathlib/MeasureTheory/Measure/ProbabilityMeasure.lean,Mathlib/Topology/ContinuousMap/CompactlySupported.lean |
5 |
9 |
['FormulaRabbit81', 'YaelDillies', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
6-46062 6 days ago |
6-53340 6 days ago |
0-474 7 minutes |
| 30504 |
grunweg author:grunweg |
feat: add custom elaborators for immersions |
And golf the fail using it, a bit. Other usage sites expose bugs or unexpected error messages...
TODO: add basic tests for basic usage
TODO: fix those errors (then try to golf further!
---
- [x] depends on: #30307
- [ ] depends on: #30356
[](https://gitpod.io/from-referrer/)
|
t-differential-geometry
merge-conflict
|
688/23 |
Mathlib.lean,Mathlib/Geometry/Manifold/IsImmersionEmbedding.lean,Mathlib/Geometry/Manifold/LocalSourceTargetProperty.lean,Mathlib/Geometry/Manifold/Notation.lean,MathlibTest/DifferentialGeometry/Notation.lean,docs/references.bib |
6 |
4 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
4-81612 4 days ago |
4-81614 4 days ago |
0-13 13 seconds |
| 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
|
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 |
4-72458 4 days ago |
4-72460 4 days ago |
0-562 9 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
- [x] depends on: #22556
- [x] depends on: #22547
- [x] 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
WIP
|
42432/502 |
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 |
299 |
n/a |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
3-75430 3 days ago |
unknown |
unknown |
| 30989 |
kckennylau author:kckennylau |
feat(RingTheory): Teichmuller map |
Let `R` be an `I`-adically complete ring, and `p` be a prime number with `p ∈ I`. This PR constructs the Teichmüller map `Perfection (R ⧸ I) p →*₀ R` such that it composed with the quotient map `R →+* R ⧸ I` is the "0-th coefficient" map `Perfection (R ⧸ I) p →+* R ⧸ I`.
This generalises the existing [PreTilt.untilt](https://leanprover-community.github.io/mathlib4_docs/Mathlib/RingTheory/Perfectoid/Untilt.html#PreTilt.untilt).
I have also moved `Mathlib/LinearAlgebra/SModEq` to a folder to be `/SModEq/Basic.lean`, because I needed to add some lemmas to `/SModEq/Prime.lean`; I also added a lemma to the end of `/Basic.lean` called `ideal`.
---
In order to try to artificially minimise the diff count, I have made #30990 which only moves the file `SModEq`.
- [x] depends on: #30990
- [x] depends on: #31193
- [x] depends on: #31195
[](https://gitpod.io/from-referrer/)
|
merge-conflict
awaiting-author
|
207/112 |
Mathlib.lean,Mathlib/LinearAlgebra/SModEq/Basic.lean,Mathlib/LinearAlgebra/SModEq/Prime.lean,Mathlib/RingTheory/Perfectoid/Untilt.lean,Mathlib/RingTheory/Teichmuller.lean |
5 |
38 |
['erdOne', 'github-actions', 'jjdishere', 'kbuzzard', 'kckennylau', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'pechersky'] |
nobody |
3-30232 3 days ago |
3-30233 3 days ago |
20-9220 20 days |
| 32242 |
vihdzp author:vihdzp |
feat: missing instances for `OrderDual`/`Lex`/`Colex` |
---
The `Nonempty` and `Inhabited` instances for `OrderDual` exist in `Order.Basic` already.
[](https://gitpod.io/from-referrer/)
|
t-order
merge-conflict
|
14/16 |
Mathlib/Order/Synonym.lean |
1 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
3-1751 3 days ago |
3-1752 3 days ago |
2-55967 2 days |
| 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 |
2-73323 2 days ago |
2-73323 2 days ago |
0-0 0 seconds |
| 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 |
2-73303 2 days ago |
2-73303 2 days ago |
0-0 0 seconds |
| 29435 |
sgouezel author:sgouezel |
WIP: typeclass experiment |
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
WIP
label:t-algebra$ |
33/7 |
Mathlib/Algebra/QuadraticAlgebra.lean,Mathlib/Algebra/Ring/Defs.lean,Mathlib/GroupTheory/GroupAction/Hom.lean |
3 |
6 |
['eric-wieser', 'github-actions', 'leanprover-bot', 'mathlib4-merge-conflict-bot', 'sgouezel'] |
nobody |
2-73287 2 days ago |
2-73287 2 days ago |
0-0 0 seconds |
| 27703 |
vihdzp author:vihdzp |
feat: `le_of_forall_ne` et. al |
---
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
merge-conflict
awaiting-author
|
30/0 |
Mathlib/Order/Basic.lean |
1 |
12 |
['JovanGerb', 'eric-wieser', 'github-actions', 'mathlib4-merge-conflict-bot', 'pechersky', 'vihdzp'] |
pechersky assignee:pechersky |
2-60085 2 days ago |
2-62293 2 days ago |
12-17525 12 days |
| 31950 |
callesonne author:callesonne |
feat(CategoryTheory/Product/Basic): make `Hom` into a 1-field structure |
This should help unification.
---
[](https://gitpod.io/from-referrer/)
|
t-category-theory
merge-conflict
WIP
|
80/68 |
Mathlib/CategoryTheory/Comma/Basic.lean,Mathlib/CategoryTheory/Discrete/SumsProducts.lean,Mathlib/CategoryTheory/Functor/Currying.lean,Mathlib/CategoryTheory/Functor/CurryingThree.lean,Mathlib/CategoryTheory/Functor/Hom.lean,Mathlib/CategoryTheory/Groupoid.lean,Mathlib/CategoryTheory/Limits/FormalCoproducts.lean,Mathlib/CategoryTheory/Monoidal/Category.lean,Mathlib/CategoryTheory/MorphismProperty/Basic.lean,Mathlib/CategoryTheory/Products/Associator.lean,Mathlib/CategoryTheory/Products/Basic.lean,Mathlib/CategoryTheory/Products/Unitor.lean,Mathlib/CategoryTheory/Sums/Products.lean,Mathlib/CategoryTheory/Yoneda.lean |
14 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
2-54685 2 days ago |
2-54686 2 days ago |
0-6 6 seconds |
| 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
merge-conflict
awaiting-author
label:t-algebra$ |
270/5 |
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/LinearAlgebra/TensorPower/Symmetric.lean,Mathlib/RingTheory/PiTensorProduct.lean,Mathlib/SetTheory/Cardinal/Finite.lean |
10 |
30 |
['eric-wieser', 'github-actions', 'joelriou', 'leanprover-community-bot-assistant', 'mathlib4-merge-conflict-bot', 'riccardobrasca'] |
mattrobball assignee:mattrobball |
2-51832 2 days ago |
16-1515 16 days ago |
97-36349 97 days |
| 31671 |
vasnesterov author:vasnesterov |
feat: `norm_num` extension for `IsSquare` via `Irrational` |
1. Add `evalIrrational`: `norm_num` extension for disproving `Irrational x` for rational `x`.
2. Add `evalIsSquare`: `norm_num` extension for deciding `IsSquare x` for rational `x`. It rewrites the goal as `0 ≤ x ∧ ¬ Irrational √x` and reuses `evalIrrationalSqrt` to prove/disprove it.
---
[](https://gitpod.io/from-referrer/)
|
t-meta
merge-conflict
WIP
|
124/14 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/NormNum/Irrational.lean,Mathlib/Tactic/NormNum/IsSquare.lean,MathlibTest/norm_num_ext.lean,scripts/noshake.json |
6 |
7 |
['bryangingechen', 'github-actions', 'mathlib4-merge-conflict-bot', 'urkud', 'vasnesterov', 'yury-harmonic'] |
nobody |
2-43535 2 days ago |
18-65985 18 days ago |
0-1534 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/)
|
merge-conflict |
2/0 |
scripts/bench/fake-root/lib/lean/libleanshared.so,scripts/bench/run |
2 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
2-39817 2 days ago |
2-39817 2 days ago |
0-0 0 seconds |
| 31110 |
bryangingechen author:bryangingechen |
ci: don't delete merged branches |
This will only affect PRs that are not from forks (e.g. this one).
The motivation is that #30913 was closed automatically due to its target branch deleted after #30912 was merged. See also [#PR reviews > #30913 feat(Computability/Language):add subtraction notation @ 💬](https://leanprover.zulipchat.com/#narrow/channel/144837-PR-reviews/topic/.2330913.20feat.28Computability.2FLanguage.29.3Aadd.20subtraction.20notation/near/548052556).
Looking at the history, it looks like this option hasn't been changed since we added bors to mathlib3: https://github.com/leanprover-community/mathlib3/pull/2322
---
[](https://gitpod.io/from-referrer/)
|
CI
merge-conflict
awaiting-author
|
1/1 |
bors.toml |
1 |
4 |
['bryangingechen', 'eric-wieser', 'github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
2-36096 2 days ago |
2-36097 2 days ago |
0-64677 17 hours |
| 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.
---
- [x] depends on: #27362
- [x] depends on: #27361
- [x] depends on: #27363
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
awaiting-author
label:t-algebra$ |
142/1 |
Mathlib.lean,Mathlib/RepresentationTheory/Homological/FiniteCyclic.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/FiniteCyclic.lean |
3 |
8 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'riccardobrasca'] |
riccardobrasca assignee:riccardobrasca |
1-75426 1 day ago |
37-71896 1 month ago |
24-7427 24 days |
| 30122 |
xroblot author:xroblot |
Development branch (1) |
---
|
merge-conflict
WIP
|
3034/7 |
Mathlib.GaloisTower.lean,Mathlib/AddCharTrace.lean,Mathlib/Cyclotomic.lean,Mathlib/Data/Nat/Digits/Lemmas.lean,Mathlib/GaussSum.lean,Mathlib/KroneckerWeber_Blueprint.lean,Mathlib/Misc.lean,Mathlib/NumberTheory/MulChar/Basic.lean,Mathlib/NumberTheory/NumberField/Cyclotomic/Ideal.lean,Mathlib/NumberTheory/RamificationInertia/Galois.lean,Mathlib/RingTheory/Ideal/GoingUp.lean,Mathlib/RingTheory/Ideal/Int.lean,Mathlib/StickElt.lean,Mathlib/Teichmuller.lean |
14 |
9 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
1-66013 1 day ago |
1-66014 1 day ago |
0-12 12 seconds |
| 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.
---
Zulip announcement: [#announce > New tactic: `compute_asymptotics`](https://leanprover.zulipchat.com/#narrow/channel/113486-announce/topic/New.20tactic.3A.20.60compute_asymptotics.60/with/538639418)
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, 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
* Implement eventual zeroness oracle.
* Support different domains in `compute_limit` as well.
* 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.
- [x] depends on: #31047
- [x] depends on: #28874
[](https://gitpod.io/from-referrer/)
|
t-analysis
t-meta
merge-conflict
WIP
|
17665/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/ConvertDomain.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,scripts/README.md,scripts/migrate_to_fork.py,scripts/noshake.json |
53 |
7 |
['grunweg', 'mathlib4-dependent-issues-bot', 'ocfnash', 'vasnesterov'] |
nobody |
1-64034 1 day ago |
28-42530 28 days ago |
0-54 54 seconds |
| 30966 |
gasparattila author:gasparattila |
refactor: disable `simp` in `measurability` |
---
[](https://gitpod.io/from-referrer/)
|
merge-conflict |
5/3 |
Mathlib/MeasureTheory/MeasurableSpace/Constructions.lean,Mathlib/MeasureTheory/MeasurableSpace/Defs.lean,Mathlib/MeasureTheory/Measure/MeasureSpaceDef.lean,Mathlib/MeasureTheory/Measure/Typeclasses/SFinite.lean,Mathlib/Tactic/Measurability.lean |
5 |
8 |
['github-actions', 'grunweg', 'leanprover-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
1-62431 1 day ago |
1-62432 1 day ago |
0-0 0 seconds |
| 32210 |
ADedecker author:ADedecker |
feat: iteratedFDeriv as a linear map on test functions |
Add `TestFunction.iteratedFDeriv[WithOrder]LM`, analogous to [ContDiffMapSupportedIn.iteratedFDerivWithOrderLM](https://leanprover-community.github.io/mathlib4_docs/Mathlib/Analysis/Distribution/ContDiffMapSupportedIn.html#ContDiffMapSupportedIn.iteratedFDerivWithOrderLM) and [ContDiffMapSupportedIn.iteratedFDerivLM](https://leanprover-community.github.io/mathlib4_docs/Mathlib/Analysis/Distribution/ContDiffMapSupportedIn.html#ContDiffMapSupportedIn.iteratedFDerivLM)
---
Co-authored-by: @luigi-massacci
[](https://gitpod.io/from-referrer/)
|
t-analysis
merge-conflict
|
109/2 |
Mathlib/Analysis/Distribution/TestFunction.lean |
1 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
1-39568 1 day ago |
3-75652 3 days ago |
6-63454 6 days |
| 32328 |
ADedecker author:ADedecker |
feat: template for distributions and their API |
---
[](https://gitpod.io/from-referrer/)
|
large-import
t-analysis
merge-conflict
|
888/5 |
Mathlib.lean,Mathlib/Analysis/Distribution/ContDiffMapSupportedIn.lean,Mathlib/Analysis/Distribution/Distribution.lean,Mathlib/Analysis/Distribution/TestFunction.lean |
4 |
n/a |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
1-39564 1 day ago |
unknown |
unknown |
| 32401 |
ADedecker author:ADedecker |
feat: monotonicity of D^n(U) in n and in U as CLMs |
---
[](https://gitpod.io/from-referrer/)
|
t-analysis
merge-conflict
|
176/3 |
Mathlib/Analysis/Distribution/ContDiffMapSupportedIn.lean,Mathlib/Analysis/Distribution/TestFunction.lean |
2 |
n/a |
['ADedecker', 'github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
1-39059 1 day ago |
unknown |
unknown |
| 30439 |
plp127 author:plp127 |
feat: `norm_num` extension for `IsSquare` on `Nat`, `Int`, `Rat` |
Write a `norm_num` extension to evaluate `IsSquare` for `Nat`, `Int`, `Rat`.
---
[](https://gitpod.io/from-referrer/)
|
t-meta
merge-conflict
awaiting-author
|
152/1 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/NormNum/IsSquare.lean,MathlibTest/norm_num_ext.lean |
4 |
15 |
['Rob23oba', 'dwrensha', 'github-actions', 'mathlib4-merge-conflict-bot', 'plp127', 'vasnesterov', 'yury-harmonic'] |
dwrensha assignee:dwrensha |
1-12438 1 day ago |
16-69 16 days ago |
35-85557 35 days |
| 30711 |
kim-em author:kim-em |
experiment: which `omega` can not be replaced with `grind`? |
|
merge-conflict |
1/0 |
lakefile.lean |
1 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
0-79591 22 hours ago |
0-79591 22 hours ago |
0-0 0 seconds |
| 30712 |
kim-em author:kim-em |
experiment: which `linarith` can not be replaced with `grind`? |
|
merge-conflict |
1/0 |
lakefile.lean |
1 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
0-79589 22 hours ago |
0-79590 22 hours ago |
0-0 0 seconds |
| 30718 |
kim-em author:kim-em |
experiment: merge rewrites |
|
t-meta
merge-conflict
|
1/0 |
lakefile.lean |
1 |
3 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
0-79588 22 hours ago |
0-79589 22 hours ago |
0-0 0 seconds |
| 30720 |
kim-em author:kim-em |
experiment: merge with subsequent grind |
|
merge-conflict |
1/0 |
lakefile.lean |
1 |
2 |
['github-actions', 'mathlib4-merge-conflict-bot'] |
nobody |
0-79586 22 hours ago |
0-79587 22 hours ago |
0-0 0 seconds |
| 32419 |
kim-em author:kim-em |
fix(scripts/lint-style): improve Mathlib.Init import error messages |
## Summary
Improve the `checkInitImports` linter by:
1. Accepting transitive imports (not just direct) for the `Mathlib.Init` check
2. Removing hardcoded exceptions for transitively imported files
3. Making error messages actionable with specific advice
### Two cases with different advice
1. **Transitively imported by `Mathlib.Init`** → add `import Mathlib.Tactic.Linter.Header`
2. **NOT imported by `Mathlib.Init`** → add `import Mathlib.Init`
### Example output
**Case 1: Transitively imported by Init**
```
• `Mathlib.Util.SomeFile` is transitively imported by `Mathlib.Init`.
→ Add `import Mathlib.Tactic.Linter.Header` to `Mathlib.Util.SomeFile`.
```
**Case 2: Not imported by Init**
```
• `Mathlib.Util.TestFile` is NOT imported by `Mathlib.Init`.
→ Add `import Mathlib.Init` to `Mathlib.Util.TestFile`.
```
## Implementation
Added `findTransitiveImports` helper that computes the transitive closure of imports starting from a given file. The linter now checks transitive imports instead of direct imports, eliminating the need for hardcoded exceptions.
## Context
Prompted by confusion when working on #32416 - the old error message just said files didn't import `Mathlib.Init` without explaining what to do when adding that import would create a cycle.
Discussion: https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Mathlib.2EInit.20linter.20error
## Test plan
- [x] `lake build lint-style` succeeds
- [x] `lake exe lint-style` passes (no Init import errors)
🤖 Prepared with Claude Code |
t-linter
merge-conflict
awaiting-author
|
41/16 |
scripts/lint-style.lean |
1 |
9 |
['github-actions', 'grunweg', 'kim-em', 'mathlib4-merge-conflict-bot'] |
nobody |
0-74189 20 hours ago |
0-74190 20 hours ago |
0-11150 3 hours |
| 30441 |
linesthatinterlace author:linesthatinterlace |
refactor(`Data/List/Sort`): deprecate and replace `List.Sorted` |
Deprecates `Sorted` and defines new special-case predicates to be used for preorders.
`List.Sorted` is essentially an irrelevant definition, as it is identical to List.Pairwise, and we have some results about Sorted which also always apply to Pairwise or do so under certain conditions (and vice versa). We also commonly use Sorted to talk specifically about `<` and `<=`, which can be somewhat unwieldy. As a result, this PR does the following.
### Deprecate List.Sorted
`List.Sorted` is currently just a synonym of `List.Pairwise`, but it isn't even an `abbrev`. We deprecate it here along with theorems that are just repeats from Pairwise.
### Separate out InsertionSort and MergeSort content
We extract the theorems about insertion sort and merge sort that currently exist in the context of `List.Sorted` - they are currently in the same file but I think they could go elsewhere, potentially even into `Batteries` where I think they would naturally fit - they aren't really mathematical in nature IMO.
### Define `Sorted*` predicates.
It is useful to have predicates `SortedLT`, `SortedLE`, `SortedGT` and `SortedGE`, which correspond to exactly what they sound like. These are equivalent to suitable `Pairwise` statements, but that is not how they are defined - one could equivalently define them using `IsChain`, or, as I do here, using monotonicity of `List.get`. While the latter is how they are defined, I use irreducible definitions - it is not permitted to use the definitions directly. Instead, API is provided so that you can easily move to/from monotonicity statements, Pairwise statements, and IsChain statements. You don't destructure lists directly here: to prove things from, say, (a :: b :: l).sortedLT, one probably accesses IsChain lemmas to extract things from this statement. But one can also use the monotonicty API to prove things usefully. `Data.List.Sorted` contains all of this and I think it exhibits my thinking on what should be possible.
I've actually changed my mind a couple of times on how to actually define these - one could use Pairwise, IsChain or Monotone etc. to taste - but it doesn't matter, because the API is robust enough that it changes very little once one establishes the core set of facts/equivalence between these.
### In particular, add better decidability instance
[List.decidableSorted](https://leanprover-community.github.io/mathlib4_docs/Mathlib/Data/List/Sort.html#List.decidableSorted) has the fundamental issue that `List.Sorted` seems conceptually meant for transitive relations, but the instance of Decidable it uses uses Pairwise's decidability, not IsChain's. This is a problem because the latter is O(n) and the former is O(n^2), where n is the length of the list. It's not a major deal one might think - but I think being able to efficiently check whether something is <-sorted or <=-sorted is important.
### Adapt library to changes
I think nearly everywhere we *actually use* `List.Sorted` it is in the context of (<) or (<=), so I've changed to using these specific predicates.
---
[](https://gitpod.io/from-referrer/)
|
t-data
merge-conflict
|
995/638 |
Mathlib.lean,Mathlib/AlgebraicTopology/SimplexCategory/GeneratorsRelations/NormalForms.lean,Mathlib/Analysis/Convex/BetweenList.lean,Mathlib/Analysis/Matrix/Spectrum.lean,Mathlib/Combinatorics/Young/YoungDiagram.lean,Mathlib/Data/Fin/Tuple/Sort.lean,Mathlib/Data/Finset/Sort.lean,Mathlib/Data/List/Nodup.lean,Mathlib/Data/List/NodupEquivFin.lean,Mathlib/Data/List/OfFn.lean,Mathlib/Data/List/Pairwise.lean,Mathlib/Data/List/Sort.lean,Mathlib/Data/Multiset/Sort.lean,Mathlib/Data/Nat/BitIndices.lean,Mathlib/Data/Nat/Factors.lean,Mathlib/Deprecated/Sort.lean,Mathlib/Logic/Equiv/Finset.lean,Mathlib/Logic/Equiv/Multiset.lean,Mathlib/NumberTheory/ADEInequality.lean,Mathlib/NumberTheory/Divisors.lean,Mathlib/Order/JordanHolder.lean,Mathlib/Order/RelSeries.lean,Mathlib/Order/Synonym.lean,Mathlib/SetTheory/Ordinal/Basic.lean,Mathlib/SetTheory/Ordinal/CantorNormalForm.lean,Mathlib/Tactic/Simproc/Factors.lean,Mathlib/Topology/Category/Profinite/Nobeling/Basic.lean,Mathlib/Topology/Category/Profinite/Nobeling/Span.lean |
28 |
85 |
['Vierkantor', 'github-actions', 'joelriou', 'linesthatinterlace', 'mathlib-bors', 'mathlib4-merge-conflict-bot', 'riccardobrasca', 'vihdzp'] |
Vierkantor assignee:Vierkantor |
0-71124 19 hours ago |
0-74886 20 hours ago |
36-13100 36 days |
| 32127 |
CoolRmal author:CoolRmal |
feat: use IndexedPartition.piecewise to create simple/measurable/strongly measurable functions |
The lemmas proved in this PR are needed in https://github.com/RemyDegenne/brownian-motion/pull/304.
---
[](https://gitpod.io/from-referrer/)
|
brownian
large-import
t-measure-probability
merge-conflict
|
122/4 |
Mathlib/Data/Setoid/Partition.lean,Mathlib/MeasureTheory/Function/SimpleFunc.lean,Mathlib/MeasureTheory/Function/StronglyMeasurable/Basic.lean,Mathlib/MeasureTheory/MeasurableSpace/Basic.lean |
4 |
17 |
['CoolRmal', 'EtienneC30', 'github-actions', 'hanwenzhu', 'mathlib4-merge-conflict-bot'] |
EtienneC30 assignee:EtienneC30 |
0-47953 13 hours ago |
0-47954 13 hours ago |
8-9383 8 days |
| 29203 |
Hagb author:Hagb |
feat(RingTheory/MvPolynomial/Groebner): add Gröbner basis |
Definitions:
- `MonomialOrder.IsRemainder`
- `MonomialOrder.IsGroebnerBasis`
Main theorems:
* `MonomialOrder.remainder_eq_zero_iff_mem_ideal_of_isGroebnerBasis`: Given a remainder of a polynomial on division by a Gröbner basis of an ideal, the remainder is 0 if and only if the polynomial is in the ideal.
* `MonomialOrder.isGroebnerBasis_iff_subset_ideal_and_isRemainder_zero`: A finite set of polynomials is a Gröbner basis of an ideal if and only if it is a subset of this ideal and 0 is a remainder of each member of this ideal on division by this finite set.
* `MonomialOrder.existsUnique_isRemainder_of_isGroebnerBasis`: Remainder of any polynomial on division by a Gröbner basis exists and is unique.
* `MonomialOrder.ideal_eq_span_of_isGroebnerBasis`: Gröbner basis of any ideal spans the ideal.
* `MonomialOrder.isGroebnerBasis_iff_isRemainder_sPolynomial_zero` (Buchberger Criterion): a basis of an ideal is a Gröbner basis of it if and only if 0 is a remainder of echo sPolynomial between two polynomials on the basis.
TODO:
- squeeze Non-terminal `simp`s
- add comments to explain the proof of Buchberger Criterion.
Co-authored-by: Hao Shen [3118181069@qq.com](mailto:3118181069@qq.com)
---
CC @tsuki8
Upstreamize from https://github.com/WuProver/groebner_proj.
- [x] depends on: #26039
- [x] depends on: #32336
- [ ] depends on: #32344
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
merge-conflict
awaiting-author
WIP
|
1614/3 |
Mathlib/RingTheory/MvPolynomial/Groebner.lean,Mathlib/RingTheory/MvPolynomial/Ideal.lean,Mathlib/RingTheory/MvPolynomial/MonomialOrder.lean,docs/references.bib |
4 |
13 |
['Hagb', 'SnirBroshi', 'github-actions', 'jcommelin', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
0-43704 12 hours ago |
2-75817 2 days ago |
1-17846 1 day |
| 31603 |
alreadydone author:alreadydone |
chore(Algebra): make `RatFunc` an abbrev |
I think there's no instance on `FractionRing K[X]` that shouldn't be shared by `RatFunc K`, so it's better to make the latter an abbrev. In the ongoing [Lüroth project](https://github.com/hdlean/mathlib4/pull/1/files#diff-02a084b8d8540eab8a346db8be4ba1a2b39b086bc1407125536d96adf6544544) I've been using `FractionRing K[X]` and it would be nice if we could gain direct access to `RatFunc` API (though not much is relevant, there was already one case where it's helpful), and if our results could be directly applied to RatFunc rather than going through some isomorphism boilerplate. Of course, some `IsRatFunc` predicate could also be an option (IsField + generated by one transcendental element over base field).
---
[](https://gitpod.io/from-referrer/)
|
t-algebra
RFC
merge-conflict
awaiting-author
label:t-algebra$ |
81/431 |
Mathlib/FieldTheory/Laurent.lean,Mathlib/FieldTheory/RatFunc/AsPolynomial.lean,Mathlib/FieldTheory/RatFunc/Basic.lean,Mathlib/FieldTheory/RatFunc/Defs.lean |
4 |
19 |
['Vierkantor', 'alreadydone', 'erdOne', 'github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'leanprover-radar', 'mathlib4-merge-conflict-bot', 'mattrobball'] |
erdOne assignee:erdOne |
0-34990 9 hours ago |
9-11723 9 days ago |
9-5124 9 days |
| 32425 |
kim-em author:kim-em |
feat(Linter/FlexibleLinter): generate Try this: simp only suggestions |
When the flexible linter detects a `simp` or `simp_all` (without `only`) followed by a rigid tactic, it now:
- re-runs simp in the original context to capture the used theorems
- generates an actionable "Try this: simp only [...]" suggestion that users can click to apply
This is a follow-up to #32421, which added the actionable warning message. This PR directly provides a fix.
Example output:
```
warning: 'simp' is a flexible tactic modifying '⊢'. Try 'simp?' and use the suggested 'simp only [...]'.
Note: This linter can be disabled with `set_option linter.flexible false`
---
info: Try this:
[apply] simp only [Nat.add_zero]
---
info: … and 'exact h.symm' uses '⊢'!
```
🤖 Prepared with Claude Code
-------------
- [ ] depends on: #32421
## Implementation
- Added imports for `Lean.Server.InfoUtils`, `Lean.Elab.Tactic.Simp`, and `Lean.Meta.Tactic.TryThis`
- Refactored to use `InfoTree.foldInfo` to capture `ContextInfo` needed to run MetaM code
- Uses `simpGoal` to re-run simp and get `usedTheorems`
- Uses `mkSimpOnly` to generate the suggestion syntax
- Falls back gracefully if simp re-run fails
|
t-linter
merge-conflict
|
212/81 |
Mathlib/Tactic/Linter/FlexibleLinter.lean,MathlibTest/FlexibleLinter.lean,MathlibTest/ImportHeavyFlexibleLinter.lean |
3 |
3 |
['github-actions', 'grunweg', 'mathlib4-dependent-issues-bot'] |
nobody |
0-9499 2 hours ago |
0-9500 2 hours ago |
0-10373 2 hours |
| 31242 |
plp127 author:plp127 |
feat: express filter as supremum of principal filter and free filter |
Prove a filter is free iff it is smaller than the cofinite filter. Prove that every filter decomposes as the disjoint supremum of a principal filter and a free filter.
---
- [ ] depends on: #31264
[](https://gitpod.io/from-referrer/)
|
t-order
merge-conflict
awaiting-author
|
55/0 |
Mathlib/Order/Filter/Cofinite.lean,Mathlib/Order/Lattice.lean |
2 |
7 |
['github-actions', 'jcommelin', 'kckennylau', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'plp127'] |
bryangingechen assignee:bryangingechen |
0-9267 2 hours ago |
0-9268 2 hours ago |
24-22847 24 days |
| 32198 |
kim-em author:kim-em |
feat: grind annotations for sup/inf associativity and commutativity |
## Summary
Add `grind` annotations for lattice sup/inf properties:
- `@[grind =]` on `sup_idem`, `sup_comm`, `inf_idem`, `inf_comm`
- `@[grind _=_]` on `sup_assoc`, `inf_assoc`
## Context
These annotations were originally part of the `grind_disjoint` PR but were removed because they cause a significant performance regression. For example, `Mathlib.Order.Interval.Set.LinearOrder` goes from **2.2s to 9.5s** (~4.3x slower) with these annotations present.
The slowdown occurs because these fundamental lattice lemmas get registered with grind's AC module, and since `⊔` and `⊓` are extremely pervasive (e.g., `max`/`min` expand to them), grind ends up doing excessive work on proofs that involve these operations.
## Status
This PR should remain as a draft until Leo adds the new AC matching module to grind, at which point these annotations may become unnecessary or the performance issue may be resolved.
🤖 Prepared with Claude Code |
merge-conflict |
79/53 |
Archive/Imo/Imo2001Q3.lean,Mathlib/Data/Finset/Disjoint.lean,Mathlib/Data/Set/Disjoint.lean,Mathlib/Order/BooleanAlgebra/Basic.lean,Mathlib/Order/BoundedOrder/Basic.lean,Mathlib/Order/BoundedOrder/Lattice.lean,Mathlib/Order/CompleteLattice/MulticoequalizerDiagram.lean,Mathlib/Order/Disjoint.lean,Mathlib/Order/Lattice.lean,Mathlib/Order/SupIndep.lean,MathlibTest/grind/pairwise_disjoint.lean |
11 |
1 |
['github-actions'] |
nobody |
0-9020 2 hours ago |
7-12173 7 days 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 |
513-67143 1 year ago |
513-67166 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 |
492-69 1 year ago |
504-11307 1 year ago |
0-0 0 seconds |
| 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 |
492-66 1 year ago |
542-41454 1 year ago |
0-34665 9 hours |
| 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 |
492-66 1 year ago |
513-67166 1 year ago |
0-15202 4 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 |
492-64 1 year ago |
556-3285 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 |
492-62 1 year ago |
513-67166 1 year ago |
0-0 0 seconds |
| 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 |
492-62 1 year ago |
553-64103 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 |
492-62 1 year ago |
513-67166 1 year ago |
6-59794 6 days |
| 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 |
492-61 1 year ago |
556-3285 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 |
487-56450 1 year ago |
487-56451 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 |
477-80115 1 year ago |
477-80115 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 |
476-76320 1 year ago |
476-76320 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 |
476-75793 1 year ago |
476-75793 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 |
476-75756 1 year ago |
476-75756 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 |
451-85792 1 year ago |
451-85792 1 year ago |
0-0 0 seconds |
| 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 |
439-29985 1 year 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 |
436-49657 1 year ago |
436-49657 1 year 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 |
431-17666 1 year ago |
431-17666 1 year 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 |
428-45635 1 year ago |
428-45636 1 year 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 |
428-45635 1 year ago |
428-45635 1 year 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 |
428-45634 1 year ago |
428-45634 1 year 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 |
415-17376 1 year ago |
415-17376 1 year 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 |
414-40290 1 year ago |
423-40764 1 year ago* |
423-40726 423 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 |
410-68292 1 year ago |
410-68292 1 year 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 |
397-79620 1 year ago |
397-79620 1 year 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 |
397-52353 1 year ago |
423-40875 1 year 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 |
391-52320 1 year ago |
391-52320 1 year ago |
0-0 0 seconds |
| 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 |
379-71884 1 year 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 |
376-22656 1 year ago |
376-22656 1 year 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 |
374-68077 1 year ago |
374-68077 1 year ago |
0-380 6 minutes |
| 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 |
359-70246 11 months ago |
369-47376 1 year 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 |
349-66944 11 months ago |
349-66944 11 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 |
349-58239 11 months ago |
385-38304 1 year 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 |
339-66369 11 months ago |
384-81997 1 year 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 |
336-39173 11 months ago |
336-39173 11 months ago |
0-3440 57 minutes |
| 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 |
325-66048 10 months ago |
372-74185 1 year 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 |
322-68636 10 months ago |
322-68636 10 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 |
320-53138 10 months ago |
476-76758 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 |
308-41537 10 months ago |
unknown |
unknown |
| 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 |
298-30872 9 months ago |
298-30872 9 months ago |
39-21495 39 days |
| 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 |
276-74190 9 months ago |
276-74190 9 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 |
276-15993 9 months ago |
276-15993 9 months ago |
92-44198 92 days |
| 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 |
274-75980 8 months ago |
274-75985 8 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 |
274-63241 8 months ago |
274-63241 8 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 |
272-77837 8 months ago |
272-77837 8 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 |
258-50296 8 months ago |
258-50296 8 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 |
248-82741 8 months ago |
248-82741 8 months ago |
16-16341 16 days |
| 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 |
239-67456 7 months ago |
239-67458 7 months ago |
0-2084 34 minutes |
| 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 |
239-67456 7 months ago |
239-67457 7 months ago |
0-336 5 minutes |
| 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 |
235-42802 7 months ago |
235-42804 7 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 |
234-61416 7 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 |
233-56207 7 months ago |
234-32026 7 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 |
233-9348 7 months ago |
233-11655 7 months ago* |
0-0 0 seconds* |
| 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 |
231-47861 7 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 |
231-47737 7 months ago |
294-44760 9 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 |
231-41958 7 months ago |
231-41958 7 months ago |
0-790 13 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 |
216-2826 7 months ago |
216-2826 7 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 |
216-1642 7 months ago |
216-1642 7 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 |
216-1326 7 months ago |
216-1326 7 months ago |
7-61243 7 days |
| 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 |
213-35161 6 months ago |
213-35166 6 months ago |
0-179 2 minutes |
| 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 |
210-32424 6 months ago |
210-32856 6 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 |
209-41870 6 months ago |
384-84531 1 year ago |
0-602 10 minutes |
| 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 |
189-56468 6 months ago |
189-56469 6 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 |
172-60049 5 months ago |
172-60645 5 months ago |
0-136 2 minutes |
| 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 |
168-82204 5 months ago |
384-84530 1 year 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 |
161-2259 5 months ago |
384-84534 1 year 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 |
160-84633 5 months ago |
384-84532 1 year 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 |
160-84629 5 months ago |
unknown |
unknown |
| 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 |
153-11900 5 months ago |
153-11900 5 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 |
153-11770 5 months ago |
153-11771 5 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 |
153-11768 5 months ago |
153-11769 5 months ago |
0-2 2 seconds |
| 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 |
143-10465 4 months ago |
365-42247 1 year ago |
22-67320 22 days |
| 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 |
133-79474 4 months ago |
133-79474 4 months 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 |
132-22643 4 months ago |
132-22644 4 months ago |
0-333 5 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 |
125-58056 4 months ago |
125-58057 4 months ago |
0-0 0 seconds |
| 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 |
122-79113 4 months ago |
122-79113 4 months 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 |
122-79104 4 months ago |
122-79104 4 months 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 |
122-79094 4 months ago |
122-79094 4 months ago |
0-0 0 seconds |
| 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 |
121-81221 3 months ago |
121-81221 3 months 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 |
121-81173 3 months ago |
121-81173 3 months ago |
0-3552 59 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 |
113-7079 3 months ago |
113-7080 3 months 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 |
113-6954 3 months ago |
113-6955 3 months ago |
0-1 1 second |
| 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 |
111-54934 3 months ago |
507-26487 1 year ago |
7-77799 7 days |
| 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 |
108-9737 3 months ago |
108-9738 3 months ago |
0-35689 9 hours |
| 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 |
107-8270 3 months ago |
107-8270 3 months ago |
0-21 21 seconds |
| 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 |
105-61572 3 months ago |
386-66241 1 year ago |
0-0 0 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 |
105-46245 3 months ago |
105-46246 3 months ago |
43-26015 43 days |
| 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 |
104-10863 3 months ago |
104-10863 3 months ago |
0-1808 30 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 |
103-72447 3 months ago |
237-7997 7 months ago* |
0-0 0 seconds* |
| 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 |
102-62269 3 months ago |
102-62269 3 months ago |
1-48447 1 day |
| 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 |
98-65832 3 months ago |
98-65833 3 months 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 |
98-65831 3 months ago |
98-65832 3 months 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 |
98-65830 3 months ago |
98-65831 3 months ago |
0-45 45 seconds |
| 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 |
98-38041 3 months ago |
98-38042 3 months 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 |
98-37916 3 months 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 |
98-37914 3 months 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 |
98-37913 3 months 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 |
95-42648 3 months ago |
95-42649 3 months ago |
0-5139 1 hour |
| 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 |
94-78108 3 months ago |
94-78109 3 months ago |
11-15676 11 days |
| 27707 |
FLDutchmann author:FLDutchmann |
feat(NumberTheory/SelbergSieve): define Selberg's weights and prove basic results. |
This PR continues the work from #23635.
Original PR: https://github.com/leanprover-community/mathlib4/pull/23635
- [ ] 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 |
94-44758 3 months ago |
94-44759 3 months 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 |
94-44757 3 months ago |
94-44758 3 months ago |
0-26 26 seconds |
| 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 |
93-30240 3 months ago |
93-30241 3 months ago |
0-0 0 seconds |
| 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 |
87-39108 2 months ago |
87-39108 2 months ago |
0-309 5 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 |
85-84653 2 months ago |
85-84654 2 months ago |
0-705 11 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 |
84-52348 2 months ago |
84-52349 2 months ago |
9-60153 9 days |
| 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 |
83-54182 2 months ago |
83-54182 2 months 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 |
83-54059 2 months ago |
83-54060 2 months ago |
0-3098 51 minutes |
| 27950 |
alreadydone author:alreadydone |
feat(MonoidAlgebra): criteria for `single` to be a unit, irreducible or prime |
---
- [ ] depends on: #27936
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
blocked-by-other-PR
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 |
77-70118 2 months ago |
120-30026 3 months ago |
0-53 53 seconds |
| 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/)
|
merge-conflict
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 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
75-72253 2 months ago |
75-72253 2 months ago |
0-2904 48 minutes |
| 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
|
439/22 |
Mathlib.lean,Mathlib/AlgebraicGeometry/AffineScheme.lean,Mathlib/AlgebraicGeometry/AlgebraicCycle.lean,Mathlib/AlgebraicGeometry/Properties.lean,Mathlib/AlgebraicGeometry/Scheme.lean,Mathlib/Topology/LocallyFinsupp.lean |
6 |
6 |
['Raph-DG', 'github-actions', 'joelriou', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
70-83018 2 months ago |
122-79371 4 months ago |
0-366 6 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
merge-conflict
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 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
66-54120 2 months ago |
66-54121 2 months 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
merge-conflict
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 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
66-54118 2 months ago |
66-54119 2 months 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
merge-conflict
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 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
66-54116 2 months ago |
66-54117 2 months 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
merge-conflict
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 |
66-53991 2 months 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
merge-conflict
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 |
66-53989 2 months 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
merge-conflict
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 |
66-53988 2 months 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
merge-conflict
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 |
66-53986 2 months 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
merge-conflict
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 |
66-53984 2 months 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
merge-conflict
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 |
4 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
66-53983 2 months ago |
66-53984 2 months ago |
0-1017 16 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
merge-conflict
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 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
66-17155 2 months ago |
66-17155 2 months ago |
0-0 0 seconds |
| 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
merge-conflict
blocked-by-other-PR
|
438/0 |
Mathlib/CategoryTheory/Limits/Shapes/Pullback/Categorical/CatCospanTransform.lean |
1 |
5 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
64-80388 2 months ago |
64-80389 2 months ago |
0-838 13 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: #28796
- [ ] depends on: #28853
- [x] 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.
- [x] 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
blocked-by-other-PR
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 |
4 |
['github-actions', 'grunweg', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] |
nobody |
63-84042 2 months ago |
64-251 2 months ago |
0-0 0 seconds |
| 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
---
- [ ] depends on: #26985
[](https://gitpod.io/from-referrer/)
|
t-analysis
merge-conflict
blocked-by-other-PR
|
271/123 |
Mathlib/Analysis/Calculus/Implicit.lean,docs/1000.yaml,docs/overview.yaml,docs/undergrad.yaml |
4 |
4 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
63-76145 2 months ago |
63-76146 2 months ago |
23-28425 23 days |
| 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.
---
- [x] depends on: #27361
- [x] depends on: #27362
- [x] 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 |
63-59103 2 months ago |
103-59002 3 months ago |
0-351 5 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
merge-conflict
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 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
63-45260 2 months ago |
63-45260 2 months ago |
0-537 8 minutes |
| 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
merge-conflict
blocked-by-other-PR
|
942/9 |
Mathlib.lean,Mathlib/AlgebraicTopology/SimplexCategory/GeneratorsRelations/Equivalence.lean,Mathlib/AlgebraicTopology/SimplexCategory/GeneratorsRelations/NormalForms.lean |
3 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
61-80764 2 months ago |
61-80765 2 months ago |
0-2 2 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 |
60-31664 1 month ago |
142-33733 4 months ago |
0-1386 23 minutes |
| 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
- [x] 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 |
59-64715 1 month ago |
116-57918 3 months ago |
0-22127 6 hours |
| 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
merge-conflict
blocked-by-other-PR
WIP
|
287/0 |
Mathlib.lean,Mathlib/Geometry/Manifold/Instances/Sphere.lean,Mathlib/Geometry/Manifold/Orientable.lean |
3 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
57-62454 1 month ago |
57-62455 1 month ago |
0-0 0 seconds |
| 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
merge-conflict
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 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
55-76136 1 month ago |
55-76137 1 month ago |
0-1600 26 minutes |
| 29282 |
Jlh18 author:Jlh18 |
feat(CategoryTheory): HasColimits instance on Grpd |
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
merge-conflict
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 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
55-59599 1 month ago |
78-76012 2 months ago |
0-396 6 minutes |
| 29387 |
mans0954 author:mans0954 |
feat(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
merge-conflict
blocked-by-other-PR
|
133/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 |
6 |
5 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
51-17030 1 month ago |
51-17031 1 month ago |
0-2474 41 minutes |
| 30610 |
grunweg author:grunweg |
feat: yet another lemma about differentiability of parametric integrals |
From sphere-eversion.
---
TODO: explicitly make Floris a co-author again
- [ ] depends on: #30608
- [ ] depends on: #30612
[](https://gitpod.io/from-referrer/)
|
t-analysis
blocked-by-other-PR
|
193/0 |
Mathlib/Analysis/Calculus/ParametricIntegral.lean |
1 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
49-57126 1 month ago |
49-57128 1 month ago |
0-7778 2 hours |
| 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
merge-conflict
blocked-by-other-PR
|
37/5 |
Mathlib/AlgebraicTopology/FundamentalGroupoid/Basic.lean,Mathlib/AlgebraicTopology/FundamentalGroupoid/SimplyConnected.lean |
2 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
47-48715 1 month ago |
47-48715 1 month ago |
0-2854 47 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
merge-conflict
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 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
47-48713 1 month ago |
47-48714 1 month ago |
0-23 23 seconds |
| 16210 |
astrainfinita author:astrainfinita |
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 |
['astrainfinita', 'github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot'] |
nobody |
47-9337 1 month ago |
458-45622 1 year ago |
0-0 0 seconds |
| 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
- [ ] depends on: #30038
- [ ] depends on: #30039
- [ ] depends on: #30042
[](https://gitpod.io/from-referrer/)
|
merge-conflict
blocked-by-other-PR
|
290/196 |
Archive/Imo/Imo1988Q6.lean,Archive/ZagierTwoSquares.lean,Counterexamples/Phillips.lean,Mathlib/Algebra/Group/Action/Pointwise/Set/Basic.lean,Mathlib/Algebra/Group/Pointwise/Finset/Basic.lean,Mathlib/Algebra/Group/Pointwise/Set/Basic.lean,Mathlib/Algebra/Group/Pointwise/Set/ListOfFn.lean,Mathlib/Algebra/Module/ZLattice/Basic.lean,Mathlib/Algebra/MonoidAlgebra/Degree.lean,Mathlib/Algebra/Notation/Pi/Defs.lean,Mathlib/Algebra/Order/Module/HahnEmbedding.lean,Mathlib/Algebra/Polynomial/Basic.lean,Mathlib/Analysis/Analytic/IsolatedZeros.lean,Mathlib/Analysis/LocallyConvex/WithSeminorms.lean,Mathlib/Analysis/Oscillation.lean,Mathlib/Analysis/SpecialFunctions/Log/Basic.lean,Mathlib/Analysis/SpecialFunctions/Log/PosLog.lean,Mathlib/CategoryTheory/Galois/Basic.lean,Mathlib/Combinatorics/Colex.lean,Mathlib/Combinatorics/Enumerative/InclusionExclusion.lean,Mathlib/Combinatorics/Hall/Finite.lean,Mathlib/Combinatorics/Matroid/Dual.lean,Mathlib/Combinatorics/SimpleGraph/Clique.lean,Mathlib/Data/Analysis/Filter.lean,Mathlib/Data/Finset/BooleanAlgebra.lean,Mathlib/Data/Finset/Card.lean,Mathlib/Data/Finset/Defs.lean,Mathlib/Data/Finset/Empty.lean,Mathlib/Data/Finset/Filter.lean,Mathlib/Data/Finset/Insert.lean,Mathlib/Data/Finset/Lattice/Basic.lean,Mathlib/Data/Finset/Max.lean,Mathlib/Data/Finset/Powerset.lean,Mathlib/Data/Finset/SDiff.lean,Mathlib/Data/Finset/Sups.lean,Mathlib/Data/Finset/Union.lean,Mathlib/Data/Fintype/Defs.lean,Mathlib/Data/Nat/Cast/Basic.lean,Mathlib/Data/Nat/Lattice.lean,Mathlib/Data/Nat/PrimeFin.lean,Mathlib/Data/Real/Archimedean.lean,Mathlib/Data/Set/Basic.lean,Mathlib/Data/Set/Insert.lean,Mathlib/Data/Set/Operations.lean,Mathlib/Data/Set/Prod.lean,Mathlib/GroupTheory/GroupAction/MultiplePrimitivity.lean,Mathlib/LinearAlgebra/AffineSpace/AffineSubspace/Defs.lean,Mathlib/LinearAlgebra/Multilinear/Basic.lean,Mathlib/LinearAlgebra/RootSystem/Base.lean,Mathlib/MeasureTheory/Constructions/BorelSpace/Order.lean,Mathlib/MeasureTheory/Constructions/Cylinders.lean,Mathlib/MeasureTheory/Constructions/Polish/Basic.lean,Mathlib/MeasureTheory/Covering/Vitali.lean,Mathlib/MeasureTheory/Function/SimpleFunc.lean,Mathlib/MeasureTheory/Measure/Restrict.lean,Mathlib/MeasureTheory/Measure/Typeclasses/Finite.lean,Mathlib/MeasureTheory/SetAlgebra.lean,Mathlib/NumberTheory/AbelSummation.lean,Mathlib/NumberTheory/Divisors.lean,Mathlib/NumberTheory/ModularForms/DedekindEta.lean,Mathlib/Order/CompactlyGenerated/Basic.lean,Mathlib/Order/CompleteLatticeIntervals.lean,Mathlib/Order/Interval/Finset/Defs.lean,Mathlib/Order/Interval/Set/Defs.lean,Mathlib/Order/LiminfLimsup.lean,Mathlib/Order/PartialSups.lean,Mathlib/Order/SetNotation.lean,Mathlib/Order/UpperLower/Basic.lean,Mathlib/Probability/Moments/ComplexMGF.lean,Mathlib/Probability/ProductMeasure.lean,Mathlib/RingTheory/HahnSeries/Summable.lean,Mathlib/RingTheory/Nilpotent/Defs.lean,Mathlib/Topology/Algebra/ProperAction/ProperlyDiscontinuous.lean,Mathlib/Topology/Bornology/BoundedOperation.lean,Mathlib/Topology/Bornology/Constructions.lean,Mathlib/Topology/Compactness/Compact.lean,Mathlib/Topology/Compactness/Lindelof.lean,Mathlib/Topology/Connected/Clopen.lean,Mathlib/Topology/ContinuousMap/BoundedCompactlySupported.lean,Mathlib/Topology/EMetricSpace/BoundedVariation.lean,Mathlib/Topology/GDelta/MetrizableSpace.lean,Mathlib/Topology/JacobsonSpace.lean,Mathlib/Topology/Order/Compact.lean,Mathlib/Topology/Order/HullKernel.lean,Mathlib/Topology/Perfect.lean,Mathlib/Topology/Sets/CompactOpenCovered.lean,MathlibTest/push.lean |
87 |
7 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
45-41805 1 month ago |
50-64877 1 month ago |
4-45292 4 days |
| 30658 |
grunweg author:grunweg |
chore: rebase and continuation of #26926 (more spacing fixes) |
---
- [x] depends on: #30663
- [x] depends on: #30685
- [x] depends on: #30687
- [x] depends on: #30688
- [x] depends on: #30689
- [ ] depends on: #30690
- [x] depends on: #30691
- [x] depends on: #30723
- [x] depends on: #30724
- [x] depends on: #30725
After that, virtually all whitespace changes are Damiano's, so I'll split those into nice pieces, review and maintainer merge.
[](https://gitpod.io/from-referrer/)
|
large-import
merge-conflict
blocked-by-other-PR
|
2771/685 |
Mathlib/Algebra/Category/ModuleCat/ChangeOfRings.lean,Mathlib/Algebra/Category/Ring/Basic.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/Defs.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/CategoryTheory/Limits/Shapes/BinaryProducts.lean,Mathlib/CategoryTheory/Monoidal/Action/Basic.lean,Mathlib/CategoryTheory/Yoneda.lean,Mathlib/Combinatorics/SimpleGraph/Regularity/Uniform.lean,Mathlib/Combinatorics/SimpleGraph/Triangle/Removal.lean,Mathlib/Computability/TuringMachine.lean,Mathlib/Control/ULiftable.lean,Mathlib/Data/EReal/Operations.lean,Mathlib/Data/Fin/Fin2.lean,Mathlib/Data/Fin/Tuple/Curry.lean,Mathlib/Data/Fin/Tuple/Embedding.lean,Mathlib/Data/Finmap.lean,Mathlib/Data/Finset/Card.lean,Mathlib/Data/Finset/Insert.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/Destutter.lean,Mathlib/Data/List/Nodup.lean,Mathlib/Data/List/Perm/Basic.lean,Mathlib/Data/List/Rotate.lean,Mathlib/Data/List/Sort.lean,Mathlib/Data/List/TakeWhile.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/ChineseRemainder.lean,Mathlib/Data/Nat/Choose/Basic.lean,Mathlib/Data/Nat/Choose/Mul.lean,Mathlib/Data/Nat/Factorial/SuperFactorial.lean,Mathlib/Data/Nat/Find.lean,Mathlib/Data/Nat/Init.lean,Mathlib/Data/Nat/Log.lean,Mathlib/Data/Nat/Sqrt.lean,Mathlib/Data/Num/Bitwise.lean,Mathlib/Data/Option/Basic.lean,Mathlib/Data/PSigma/Order.lean,Mathlib/Data/Part.lean,Mathlib/Data/Prod/Basic.lean,Mathlib/Data/Seq/Computation.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/Data/Vector/MapLemmas.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/FreeGroup/Reduce.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/Perm/Centralizer.lean,Mathlib/GroupTheory/Perm/Cycle/Concrete.lean,Mathlib/GroupTheory/PushoutI.lean,Mathlib/GroupTheory/SpecificGroups/Dihedral.lean,Mathlib/GroupTheory/SpecificGroups/Quaternion.lean,Mathlib/LinearAlgebra/Alternating/Basic.lean,Mathlib/LinearAlgebra/BilinearForm/TensorProduct.lean,Mathlib/LinearAlgebra/CliffordAlgebra/EvenEquiv.lean,Mathlib/LinearAlgebra/CliffordAlgebra/Prod.lean,Mathlib/LinearAlgebra/Eigenspace/Matrix.lean,Mathlib/LinearAlgebra/FreeProduct/Basic.lean |
201 |
4 |
['github-actions', 'grunweg', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
42-77733 1 month ago |
44-85596 1 month ago |
0-10092 2 hours |
| 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
merge-conflict
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 |
8 |
['Timeroot', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'staroperator'] |
nobody |
41-67689 1 month ago |
41-67690 1 month ago |
3-12935 3 days |
| 30898 |
vihdzp author:vihdzp |
feat: characterization of `List.splitBy` |
---
- [ ] depends on: #30892
Moved from #16837.
[](https://gitpod.io/from-referrer/)
|
large-import
t-data
merge-conflict
blocked-by-other-PR
|
118/4 |
Mathlib/Data/List/Flatten.lean,Mathlib/Data/List/SplitBy.lean |
2 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
39-40021 1 month ago |
39-40021 1 month ago |
0-2502 41 minutes |
| 30462 |
grunweg author:grunweg |
Everything I wanted about immersions |
Nothing to see yet, just for my own tracking (and for getting the cache).
Ideally, this branch would become obsolete as all dependent PRs get merged :-)
TODO: also cherry-pick the elaborators...
---
- [ ] depends on: #28865
- [ ] depends on: #30413
[](https://gitpod.io/from-referrer/)
|
merge-conflict
blocked-by-other-PR
|
1783/286 |
Mathlib.lean,Mathlib/Analysis/Calculus/ContDiff/Basic.lean,Mathlib/Analysis/Calculus/ContDiff/Defs.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/Geometry/Manifold/LocalSourceTargetProperty.lean,Mathlib/Geometry/Manifold/Notation.lean,Mathlib/Lean/Meta/Basic.lean,Mathlib/Topology/OpenPartialHomeomorph.lean,MathlibTest/DifferentialGeometry/Notation.lean,MathlibTest/DifferentialGeometry/NotationAdvanced.lean,docs/overview.yaml,docs/references.bib |
16 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
37-78694 1 month ago |
51-50670 1 month ago |
0-2567 42 minutes |
| 30303 |
franv314 author:franv314 |
chore(Topology/Instances): add deprecated module |
Add deprecated module to moved Cantor set file.
---
- [ ] depends on: #30299
[](https://gitpod.io/from-referrer/)
|
new-contributor
merge-conflict
blocked-by-other-PR
|
486/124 |
Mathlib.lean,Mathlib/Topology/Instances/CantorSet.lean,Mathlib/Topology/Instances/CantorSet/Basic.lean,Mathlib/Topology/Instances/CantorSet/Cardinality.lean,Mathlib/Topology/Instances/CantorSet/Lemmas.lean |
5 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
37-75765 1 month ago |
37-75766 1 month ago |
0-340 5 minutes |
| 30900 |
vihdzp author:vihdzp |
feat: run-length encoding |
---
- [ ] depends on: #30898
Moved from #17105.
[](https://gitpod.io/from-referrer/)
|
large-import
t-data
merge-conflict
blocked-by-other-PR
|
280/4 |
Mathlib.lean,Mathlib/Data/List/Flatten.lean,Mathlib/Data/List/RunLength.lean,Mathlib/Data/List/SplitBy.lean |
4 |
5 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'plp127'] |
nobody |
37-70760 1 month ago |
39-40020 1 month ago |
0-2418 40 minutes |
| 30579 |
smmercuri author:smmercuri |
feat : `v.adicCompletionIntegers K` is compact when `K` is a number field |
---
- [ ] depends on: #30576
[](https://gitpod.io/from-referrer/)
|
merge-conflict
blocked-by-other-PR
WIP
|
766/23 |
Mathlib/Algebra/Order/Hom/Ring.lean,Mathlib/NumberTheory/NumberField/FinitePlaces.lean,Mathlib/NumberTheory/Padics/HeightOneSpectrum.lean,Mathlib/NumberTheory/Padics/PadicIntegers.lean,Mathlib/NumberTheory/Padics/RingHoms.lean,Mathlib/NumberTheory/Padics/WithVal.lean,Mathlib/RingTheory/DedekindDomain/AdicValuation.lean,Mathlib/Topology/Algebra/Valued/WithVal.lean,Mathlib/Topology/Homeomorph/Defs.lean,Mathlib/Topology/UniformSpace/AbstractCompletion.lean,Mathlib/Topology/UniformSpace/Completion.lean |
11 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
37-13991 1 month ago |
37-13992 1 month ago |
0-13 13 seconds |
| 26377 |
Whysoserioushah author:Whysoserioushah |
feat(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 |
32-58857 1 month ago |
121-68577 3 months ago |
0-2337 38 minutes |
| 29774 |
Raph-DG author:Raph-DG |
feat(AlgebraicGeometry): Order of vanishing of elements of the function field of locally noetherian, integral schemes |
In this PR, we define the order of vanishing of elements of the function field of locally noetherian, integral schemes at points of codimension 1. This is essentially just a wrapper around the API for the order of vanishing for rings (i.e. Ring.ord and Ring.ordFrac), but I think it's good to have this too for usability.
---
- [ ] depends on: #29550
- [ ] depends on: #26735
[](https://gitpod.io/from-referrer/)
|
file-removed
merge-conflict
blocked-by-other-PR
|
770/4 |
Mathlib.lean,Mathlib/AlgebraicGeometry/OrderOfVanishing.lean,Mathlib/AlgebraicGeometry/Properties.lean,Mathlib/Order/KrullDimension.lean,Mathlib/RingTheory/DiscreteValuationRing/Basic.lean,Mathlib/RingTheory/OrderOfVanishing/Basic.lean,Mathlib/RingTheory/OrderOfVanishing/Properties.lean,Mathlib/Topology/KrullDimension.lean |
8 |
4 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
31-57857 1 month ago |
31-57858 1 month ago |
0-1197 19 minutes |
| 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
merge-conflict
blocked-by-other-PR
WIP
|
825/0 |
Mathlib.lean,Mathlib/Combinatorics/SimpleGraph/GirthDiam.lean |
2 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
31-1863 1 month ago |
31-1864 1 month ago |
0-28 28 seconds |
| 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
merge-conflict
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 |
30-24905 1 month ago |
unknown |
unknown |
| 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
merge-conflict
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 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
28-41846 28 days ago |
28-41847 28 days ago |
0-0 0 seconds |
| 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
- [x] 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 |
26-84980 26 days ago |
98-65835 3 months ago |
0-46 46 seconds |
| 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
merge-conflict
blocked-by-other-PR
WIP
|
283/0 |
Mathlib.lean,Mathlib/Combinatorics/SimpleGraph/Bipartite.lean,Mathlib/Combinatorics/SimpleGraph/Extremal/KovariSosTuran.lean |
3 |
5 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
26-83807 26 days ago |
26-83808 26 days ago |
45-15427 45 days |
| 31081 |
chrisflav author:chrisflav |
feat(RingTheory/StandardSmooth): presentation independent characterization |
We show that if `S` is of finite presentation over `R` such that `H¹(S/R) = 0` and `Ω[S⁄R]` is free on `{d sᵢ}ᵢ` for some `sᵢ : S`, then `S` is `R`-standard smooth. The converse of this is already in mathlib.
From Pi1.
---
- [ ] depends on: #31034
- [ ] depends on: #31082
- [ ] depends on: #28769
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
merge-conflict
blocked-by-other-PR
|
824/32 |
Mathlib.lean,Mathlib/Algebra/BigOperators/Finsupp/Basic.lean,Mathlib/Algebra/Group/Finsupp.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/Algebra/MvPolynomial/Eval.lean,Mathlib/Analysis/InnerProductSpace/Symmetric.lean,Mathlib/Data/Finsupp/Basic.lean,Mathlib/LinearAlgebra/Basis/Exact.lean,Mathlib/LinearAlgebra/Finsupp/Defs.lean,Mathlib/LinearAlgebra/Finsupp/Span.lean,Mathlib/LinearAlgebra/Finsupp/Supported.lean,Mathlib/LinearAlgebra/Finsupp/VectorSpace.lean,Mathlib/LinearAlgebra/LinearIndependent/Lemmas.lean,Mathlib/LinearAlgebra/Projection.lean,Mathlib/LinearAlgebra/Span/Basic.lean,Mathlib/RingTheory/Extension/Basic.lean,Mathlib/RingTheory/Extension/Cotangent/Basic.lean,Mathlib/RingTheory/Extension/Cotangent/Basis.lean,Mathlib/RingTheory/Extension/Cotangent/Free.lean,Mathlib/RingTheory/Extension/Generators.lean,Mathlib/RingTheory/Extension/Presentation/Basic.lean,Mathlib/RingTheory/Extension/Presentation/Submersive.lean,Mathlib/RingTheory/Ideal/Maps.lean,Mathlib/RingTheory/Ideal/Operations.lean,Mathlib/RingTheory/Localization/Away/Basic.lean,Mathlib/RingTheory/Smooth/StandardSmooth.lean |
29 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
24-57071 24 days ago |
34-62892 1 month ago |
0-319 5 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
merge-conflict
blocked-by-other-PR
label:t-algebra$ |
155/0 |
Mathlib.lean,Mathlib/LinearAlgebra/Matrix/GeneralLinearGroup/Basic.lean,Mathlib/LinearAlgebra/Matrix/StarAlgEquiv.lean |
3 |
4 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'themathqueen'] |
nobody |
23-42097 23 days ago |
23-42098 23 days ago |
0-412 6 minutes |
| 30258 |
imbrem author:imbrem |
feat(CategoryTheory/Monoidal): to_additive for proofs using `monoidal` |
Building on #30150, this allows us to use `@[to_additive]` on proofs containing `monoidal`, by tagging the lemmas `monoidal` outputs with `@[to_additive]` as appropriate.
Testing on my branch [`additive-monoidal-coherence`](https://github.com/imbrem/mathlib4/tree/additive-monoidal-coherence) shows that this works.
It is still future work to have either the `monoidal` tactic or a new `add_monoidal` tactic work for `AddMonoidalCategory` instances directly.
---
- [ ] depends on: #30150
[](https://gitpod.io/from-referrer/)
|
large-import
new-contributor
merge-conflict
blocked-by-other-PR
|
524/140 |
Mathlib/CategoryTheory/Monoidal/Category.lean,Mathlib/CategoryTheory/Monoidal/Discrete.lean,Mathlib/Tactic/CategoryTheory/Monoidal/Normalize.lean,Mathlib/Tactic/CategoryTheory/Monoidal/PureCoherence.lean,Mathlib/Tactic/CategoryTheory/MonoidalComp.lean,Mathlib/Tactic/ToAdditive/GuessName.lean |
6 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
22-18075 22 days ago |
22-18076 22 days ago |
0-241 4 minutes |
| 30260 |
imbrem author:imbrem |
feat(CategoryTheory/Monoidal): added CocartesianMonoidalCategory |
As discussed in #21603 and #28718; this implements chosen finite coproducts on top of `AddMonoidalCategory` as defined in #30150
---
- [ ] depends on: #30150
[](https://gitpod.io/from-referrer/)
|
large-import
new-contributor
merge-conflict
blocked-by-other-PR
|
839/125 |
Mathlib.lean,Mathlib/CategoryTheory/Monoidal/Category.lean,Mathlib/CategoryTheory/Monoidal/Cocartesian/Basic.lean,Mathlib/CategoryTheory/Monoidal/Discrete.lean,Mathlib/Tactic/ToAdditive/GuessName.lean |
5 |
4 |
['github-actions', 'imbrem', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
22-18074 22 days ago |
22-18075 22 days ago |
0-1234 20 minutes |
| 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
merge-conflict
blocked-by-other-PR
|
629/0 |
Mathlib.lean,Mathlib/Geometry/Diffeology/Basic.lean,docs/references.bib |
3 |
4 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'peabrainiac'] |
nobody |
21-78329 21 days ago |
21-78330 21 days ago |
0-785 13 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
merge-conflict
blocked-by-other-PR
|
766/0 |
Mathlib.lean,Mathlib/Geometry/Diffeology/Basic.lean,Mathlib/Geometry/Diffeology/Continuous.lean,docs/references.bib |
4 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
21-78205 21 days ago |
21-78206 21 days ago |
0-1796 29 minutes |
| 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
- [x] depends on: #29597
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
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 |
21-43860 21 days ago |
21-43860 21 days ago |
17-3113 17 days |
| 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 |
20-63327 20 days ago |
unknown |
unknown |
| 27953 |
CoolRmal author:CoolRmal |
feat(ProbabilityTheory): Conditional Jensen's Inequality |
This PR adds conditional Jensen's inequality.
---
- [ ] depends on: #31180
- [ ] depends on: #31411
- [ ] depends on: #31399
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-measure-probability
merge-conflict
blocked-by-other-PR
|
462/10 |
Mathlib.lean,Mathlib/Analysis/LocallyConvex/Separation.lean,Mathlib/MeasureTheory/Function/ConditionalExpectation/Basic.lean,Mathlib/MeasureTheory/Function/ConditionalExpectation/CondJensen.lean,Mathlib/MeasureTheory/MeasurableSpace/Constructions.lean |
5 |
8 |
['CoolRmal', 'EtienneC30', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
sgouezel assignee:sgouezel |
19-59868 19 days ago |
19-59869 19 days ago |
27-80190 27 days |
| 30640 |
SnirBroshi author:SnirBroshi |
feat(Combinatorics/SimpleGraph/Acyclic): a maximally acyclic graph is a tree |
Prove that a graph is maximally acyclic iff it is a tree, plus helpful theorems about bridges and acyclicity.
---
- [ ] depends on: #30570
[](https://gitpod.io/from-referrer/)
|
blocked-by-other-PR |
118/0 |
Mathlib/Combinatorics/SimpleGraph/Acyclic.lean,Mathlib/Combinatorics/SimpleGraph/Connectivity/Connected.lean |
2 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
19-20812 19 days ago |
27-51379 27 days ago |
0-627 10 minutes |
| 30399 |
kckennylau author:kckennylau |
feat(RingTheory): make HomogeneousLocalization.map take a graded ring hom |
and also make `Away.map`.
---
- [x] depends on: #30302
- [ ] depends on: #30312
[](https://gitpod.io/from-referrer/)
|
merge-conflict
blocked-by-other-PR
|
526/133 |
Mathlib.lean,Mathlib/Algebra/DirectSum/Internal.lean,Mathlib/AlgebraicGeometry/ProjectiveSpectrum/Basic.lean,Mathlib/AlgebraicGeometry/ProjectiveSpectrum/Proper.lean,Mathlib/AlgebraicGeometry/ProjectiveSpectrum/Scheme.lean,Mathlib/AlgebraicGeometry/ProjectiveSpectrum/StructureSheaf.lean,Mathlib/AlgebraicGeometry/ProjectiveSpectrum/Topology.lean,Mathlib/Data/FunLike/GradedFunLike.lean,Mathlib/RingTheory/GradedAlgebra/FiniteType.lean,Mathlib/RingTheory/GradedAlgebra/HomogeneousLocalization.lean,Mathlib/RingTheory/GradedAlgebra/RingHom.lean |
11 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
18-43309 18 days ago |
37-57476 1 month ago |
0-356 5 minutes |
| 30357 |
grunweg author:grunweg |
chore: golf using custom elaborators |
Test the elaborators on a large scale by trying them out.
Benchmarking results so far are very positive!
The elaborators mostly work very well. They do not handle products yet (that's a known issue).
Unexpected errors:
- the defeq check on the set fails in `Riemannian/Basic.lean`; TODO minimise and investigate
---
XXX: revert ContMDiffOn.smul_section_of_tsupport rename!
- [ ] depends on: #30463
[](https://gitpod.io/from-referrer/)
|
awaiting-bench
t-differential-geometry
merge-conflict
blocked-by-other-PR
|
2327/1311 |
Mathlib/Analysis/Complex/UpperHalfPlane/Manifold.lean,Mathlib/Analysis/Distribution/AEEqOfIntegralContDiff.lean,Mathlib/Geometry/Manifold/Algebra/LieGroup.lean,Mathlib/Geometry/Manifold/Algebra/Monoid.lean,Mathlib/Geometry/Manifold/Algebra/SmoothFunctions.lean,Mathlib/Geometry/Manifold/Algebra/Structures.lean,Mathlib/Geometry/Manifold/BumpFunction.lean,Mathlib/Geometry/Manifold/Complex.lean,Mathlib/Geometry/Manifold/ContMDiff/Atlas.lean,Mathlib/Geometry/Manifold/ContMDiff/Basic.lean,Mathlib/Geometry/Manifold/ContMDiff/Constructions.lean,Mathlib/Geometry/Manifold/ContMDiffMFDeriv.lean,Mathlib/Geometry/Manifold/Diffeomorph.lean,Mathlib/Geometry/Manifold/GroupLieAlgebra.lean,Mathlib/Geometry/Manifold/Instances/Icc.lean,Mathlib/Geometry/Manifold/Instances/UnitsOfNormedAlgebra.lean,Mathlib/Geometry/Manifold/IntegralCurve/Basic.lean,Mathlib/Geometry/Manifold/IntegralCurve/ExistUnique.lean,Mathlib/Geometry/Manifold/IntegralCurve/UniformTime.lean,Mathlib/Geometry/Manifold/LocalDiffeomorph.lean,Mathlib/Geometry/Manifold/MFDeriv/Atlas.lean,Mathlib/Geometry/Manifold/MFDeriv/SpecificFunctions.lean,Mathlib/Geometry/Manifold/MFDeriv/Tangent.lean,Mathlib/Geometry/Manifold/MFDeriv/UniqueDifferential.lean,Mathlib/Geometry/Manifold/Notation.lean,Mathlib/Geometry/Manifold/PartitionOfUnity.lean,Mathlib/Geometry/Manifold/Riemannian/Basic.lean,Mathlib/Geometry/Manifold/Riemannian/PathELength.lean,Mathlib/Geometry/Manifold/Sheaf/Smooth.lean,Mathlib/Geometry/Manifold/VectorBundle/Hom.lean,Mathlib/Geometry/Manifold/VectorBundle/MDifferentiable.lean,Mathlib/Geometry/Manifold/VectorBundle/Riemannian.lean,Mathlib/Geometry/Manifold/VectorBundle/SmoothSection.lean,Mathlib/Geometry/Manifold/VectorBundle/Tangent.lean,Mathlib/Geometry/Manifold/VectorField/LieBracket.lean,Mathlib/Geometry/Manifold/VectorField/Pullback.lean,Mathlib/Geometry/Manifold/WhitneyEmbedding.lean,Mathlib/NumberTheory/ModularForms/Basic.lean,Mathlib/NumberTheory/ModularForms/EisensteinSeries/MDifferentiable.lean,Mathlib/NumberTheory/ModularForms/JacobiTheta/Manifold.lean,MathlibTest/DifferentialGeometry/Notation.lean,MathlibTest/DifferentialGeometry/NotationAdvanced.lean,build.yml,small diffeo tasks-projects for newbes.md,test.lean |
45 |
10 |
['github-actions', 'grunweg', 'leanprover-bot', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
17-56457 17 days ago |
37-75765 1 month ago |
0-287 4 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
merge-conflict
blocked-by-other-PR
help-wanted
|
257/7 |
Mathlib/Control/Monad/Cont.lean,Mathlib/Data/Matrix/Auto.lean,MathlibTest/matrix_auto.lean |
3 |
8 |
['eric-wieser', 'github-actions', 'kim-em', 'leanprover-community-bot-assistant', 'mathlib4-merge-conflict-bot'] |
nobody |
16-2908 16 days ago |
16-2909 16 days ago |
0-0 0 seconds |
| 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
merge-conflict
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 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
16-2352 16 days ago |
16-2353 16 days ago |
0-37 37 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
merge-conflict
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 |
33 |
['Timeroot', 'YaelDillies', 'eric-wieser', 'github-actions', 'jcommelin', 'kbuzzard', 'kim-em', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'wmacmil'] |
nobody |
16-2221 16 days ago |
16-2222 16 days ago |
43-16103 43 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
merge-conflict
blocked-by-other-PR
|
676/0 |
Mathlib.lean,Mathlib/Computability/QueryComplexity/Basic.lean,Mathlib/Computability/QueryComplexity/Defs.lean,Mathlib/Computability/QueryComplexity/Sort.lean |
4 |
4 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
16-2212 16 days ago |
16-2213 16 days ago |
0-41 41 seconds |
| 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
merge-conflict
blocked-by-other-PR
|
215/5 |
Mathlib/ModelTheory/PartialEquiv.lean,Mathlib/ModelTheory/Substructures.lean |
2 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
16-2208 16 days ago |
16-2209 16 days ago |
0-668 11 minutes |
| 22232 |
pechersky author:pechersky |
feat(Algebra/Valued): `AdicExpansion.apprUpto` |
---
- [ ] depends on: #22231
[](https://gitpod.io/from-referrer/) |
t-topology
merge-conflict
blocked-by-other-PR
|
399/0 |
Mathlib.lean,Mathlib/Topology/Algebra/Valued/AdicExpansion.lean |
2 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
16-2066 16 days ago |
16-2067 16 days ago |
0-414 6 minutes |
| 22233 |
pechersky author:pechersky |
feat(Algebra/Valued): `AdicExpansion.evalAt` |
---
- [ ] depends on: #22231
[](https://gitpod.io/from-referrer/)
|
t-topology
merge-conflict
blocked-by-other-PR
|
488/0 |
Mathlib.lean,Mathlib/Topology/Algebra/Valued/AdicExpansion.lean |
2 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
16-2065 16 days ago |
16-2066 16 days ago |
0-412 6 minutes |
| 23460 |
Timeroot author:Timeroot |
feat: Definition of `Clone` |
Basics about Clones. Part of #20051
---
- [ ] depends on: #26329
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
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 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
16-2037 16 days ago |
16-2039 16 days ago |
65-54988 65 days |
| 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
merge-conflict
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 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
16-1745 16 days ago |
16-1746 16 days 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
merge-conflict
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 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
16-1743 16 days ago |
16-1744 16 days 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
merge-conflict
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 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
16-1741 16 days ago |
16-1742 16 days 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
merge-conflict
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 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
16-1740 16 days ago |
16-1740 16 days 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
merge-conflict
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 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
16-1738 16 days ago |
16-1739 16 days ago |
0-0 0 seconds |
| 26061 |
kckennylau author:kckennylau |
(WIP) 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)
I am currently using this PR as a hub for future PR's that will be split from this PR, so it is currently WIP.
- [ ] depends on: #30355
- [x] depends on: #30173
- [x] depends on: #30302
- [ ] depends on: #30312
- [ ] depends on: #30322
- [ ] depends on: #30334
- [ ] depends on: #30336
- [ ] depends on: #30352
- [ ] depends on: #30365
- [ ] depends on: #30367
- [ ] depends on: #30379
- [ ] depends on: #30399
- [ ] depends on: #30408
[](https://gitpod.io/from-referrer/)
|
t-algebraic-geometry
merge-conflict
blocked-by-other-PR
WIP
|
2009/0 |
Mathlib.lean,Mathlib/AlgebraicGeometry/ProjectiveSpace.lean |
2 |
16 |
['callesonne', 'erdOne', 'github-actions', 'kckennylau', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
erdOne assignee:erdOne |
16-1705 16 days ago |
16-1706 16 days ago |
110-81419 110 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
merge-conflict
blocked-by-other-PR
|
432/0 |
Mathlib.lean,Mathlib/MeasureTheory/VectorMeasure/Variation/Defs.lean,Mathlib/MeasureTheory/VectorMeasure/Variation/Lemmas.lean |
3 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
16-1560 16 days ago |
16-1561 16 days ago |
15-68781 15 days |
| 26165 |
oliver-butterley author:oliver-butterley |
feat(MeasureTheory.VectorMeasure): add lemma which shows that variation of a `ℝ≥0∞` VectorMeasure is equal to itself |
Add a lemma for the variation of a VectorMeasure which tells that if `μ` is `VectorMeasure X ℝ≥0∞` then `variation μ = μ`.
Co-authored-by: @yoh-tanimoto
- [ ] depends on: #26160
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-measure-probability
merge-conflict
blocked-by-other-PR
|
467/0 |
Mathlib.lean,Mathlib/MeasureTheory/VectorMeasure/Variation/Defs.lean,Mathlib/MeasureTheory/VectorMeasure/Variation/Lemmas.lean |
3 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
16-1559 16 days ago |
16-1560 16 days ago |
15-66224 15 days |
| 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
merge-conflict
blocked-by-other-PR
|
639/60 |
Mathlib.lean,Mathlib/FieldTheory/AxGrothendieck.lean,Mathlib/ModelTheory/FunctionalFormula.lean |
3 |
4 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
16-1518 16 days ago |
16-1519 16 days ago |
0-2300 38 minutes |
| 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$ |
446/0 |
Mathlib.lean,Mathlib/RingTheory/FilteredAlgebra/AssociatedGraded.lean |
2 |
n/a |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
16-1376 16 days 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$ |
559/0 |
Mathlib.lean,Mathlib/RingTheory/FilteredAlgebra/AssociatedGraded.lean |
2 |
n/a |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
16-1373 16 days 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$ |
665/0 |
Mathlib.lean,Mathlib/RingTheory/FilteredAlgebra/AssociatedGraded.lean |
2 |
n/a |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
16-1372 16 days 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$ |
360/0 |
Mathlib.lean,Mathlib/RingTheory/FilteredAlgebra/AssociatedGraded.lean,Mathlib/RingTheory/FilteredAlgebra/FilteredHom.lean |
3 |
4 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
16-1371 16 days ago |
16-1372 16 days 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$ |
816/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 |
16-1370 16 days 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$ |
1046/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 |
16-1369 16 days 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$ |
1196/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 |
16-1367 16 days 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$ |
516/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 |
16-1366 16 days 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$ |
715/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 |
16-1365 16 days ago |
unknown |
unknown |
| 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
merge-conflict
awaiting-author
blocked-by-other-PR
label:t-algebra$ |
257/34 |
Mathlib.lean,Mathlib/Algebra/GroupWithZero/Range.lean,Mathlib/Algebra/Order/GroupWithZero/Range.lean,Mathlib/Algebra/Order/GroupWithZero/WithZero.lean,Mathlib/RingTheory/Valuation/Basic.lean,Mathlib/RingTheory/Valuation/RankOne.lean,Mathlib/Topology/Algebra/Valued/NormedValued.lean |
7 |
15 |
['faenuccio', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'pechersky'] |
nobody |
16-1363 16 days ago |
16-1364 16 days ago |
0-117 1 minute |
| 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
merge-conflict
blocked-by-other-PR
|
299/3 |
Mathlib.lean,Mathlib/Algebra/GroupWithZero/Range.lean,Mathlib/Algebra/Order/GroupWithZero/Range.lean,Mathlib/Algebra/Order/GroupWithZero/WithZero.lean,Mathlib/Algebra/Order/Monoid/WithTop.lean,Mathlib/RingTheory/Valuation/ValueGroupIso.lean |
6 |
10 |
['faenuccio', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'pechersky'] |
faenuccio assignee:faenuccio |
16-1358 16 days ago |
16-1359 16 days ago |
10-67838 10 days |
| 27378 |
peakpoint author:peakpoint |
refactor(Geometry/Euclidean/Projection): redefine projection and reflection for affine subspaces |
This PR continues the work from #25578.
Original PR: https://github.com/leanprover-community/mathlib4/pull/25578
- [ ] depends on: #31395 |
new-contributor
t-euclidean-geometry
merge-conflict
blocked-by-other-PR
|
316/321 |
Mathlib/Analysis/Normed/Affine/Isometry.lean,Mathlib/Geometry/Euclidean/Circumcenter.lean,Mathlib/Geometry/Euclidean/Projection.lean |
3 |
10 |
['github-actions', 'jsm28', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'peakpoint'] |
nobody |
16-1209 16 days ago |
16-1210 16 days ago |
15-31228 15 days |
| 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
merge-conflict
blocked-by-other-PR
|
259/0 |
Mathlib.lean,Mathlib/Topology/FoldTrans.lean,Mathlib/Topology/Subpath.lean |
3 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
16-1055 16 days ago |
16-1056 16 days ago |
0-2340 39 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
merge-conflict
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 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
16-1044 16 days ago |
16-1044 16 days ago |
0-3692 1 hour |
| 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
merge-conflict
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 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
16-1043 16 days ago |
16-1043 16 days ago |
0-591 9 minutes |
| 29425 |
pechersky author:pechersky |
feat(NumberTheory/Padics/Torsion): `HasEnoughRootsOfUnity ℤ_[p] (p - 1)` |
---
[](https://gitpod.io/from-referrer/)
- [x] depends on: #29403
- [x] depends on: #29404
- [x] depends on: #29405
- [x] depends on: #29408
- [x] depends on: #29424
- [ ] depends on: #30989
|
t-ring-theory
merge-conflict
awaiting-author
blocked-by-other-PR
|
179/0 |
Mathlib.lean,Mathlib/NumberTheory/Padics/Torsion.lean,Mathlib/RingTheory/ZMod/Torsion.lean |
3 |
6 |
['erdOne', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'pechersky'] |
erdOne assignee:erdOne |
16-876 16 days ago |
16-877 16 days ago |
44-24953 44 days |
| 30001 |
vihdzp author:vihdzp |
feat: concept generated by set of objects/attributes |
---
- [ ] depends on: #29996
[](https://gitpod.io/from-referrer/)
|
t-order
merge-conflict
blocked-by-other-PR
|
270/99 |
Mathlib/Order/Concept.lean |
1 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
16-260 16 days ago |
16-261 16 days ago |
0-375 6 minutes |
| 30077 |
agjftucker author:agjftucker |
feat(Analysis/Calculus/ImplicitFunOfBivariate): define implicitFunOfBivariate |
In this specialization of the implicit function theorem, to an equation involving a curried bivariate function, we make assumptions on each of the partial derivatives individually. Consequently it requires import of results depending on the mean value theorem, and is sequestered to its own file apart from `Implicit.lean`.
---
- [ ] depends on: #26985
[](https://gitpod.io/from-referrer/)
|
t-analysis
merge-conflict
blocked-by-other-PR
|
264/4 |
Mathlib.lean,Mathlib/Analysis/Calculus/FDeriv/Partial.lean,Mathlib/Analysis/Calculus/Implicit.lean,Mathlib/Analysis/Calculus/ImplicitFunOfBivariate.lean |
4 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
16-247 16 days ago |
16-248 16 days ago |
0-749 12 minutes |
| 30112 |
gaetanserre author:gaetanserre |
feat(Probability.Kernel): add representation of kernel as a map of a uniform measure |
Add results about isolation of kernels randomness. In particular, it shows that one
can write a Markov kernel as the map by a deterministic of a uniform measure on `[0, 1]`.
It corresponds to Lemma 4.22 in "[Foundations of Modern Probability](https://link.springer.com/book/10.1007/978-3-030-61871-1)" by Olav Kallenberg, 2021.
---
I'm not 100% convinced by either the names of the entries or their placement. I imagine @RemyDegenne will have something to say about this.
- [ ] depends on: #27516 For a rational approximation characterization of suprema in the unit interval
[](https://gitpod.io/from-referrer/)
|
t-measure-probability
merge-conflict
blocked-by-other-PR
|
172/0 |
Mathlib.lean,Mathlib/MeasureTheory/Constructions/UnitInterval.lean,Mathlib/Probability/Kernel/Representation.lean,Mathlib/Topology/UnitInterval.lean |
4 |
5 |
['RemyDegenne', 'gaetanserre', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
16-241 16 days ago |
16-242 16 days ago |
0-318 5 minutes |
| 30230 |
CoolRmal author:CoolRmal |
feat(MeasureTheory): Basic properties of the integral against a vector measure with a bilinear form. |
Create a folder named Integral in the folder about vector measures. Define the integral of a function against a vector measure with a bilinear form, and prove that integral is a linear operator on functions, bilinear forms, and vector measures, respectively. Several useful lemmas are added into the file about variations of a vector measure (e.g. triangle inequality).
---
- [ ] depends on: #28499
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-measure-probability
merge-conflict
blocked-by-other-PR
|
1353/0 |
Mathlib.lean,Mathlib/MeasureTheory/VectorMeasure/Basic.lean,Mathlib/MeasureTheory/VectorMeasure/Integral/Basic.lean,Mathlib/MeasureTheory/VectorMeasure/Integral/L1.lean,Mathlib/MeasureTheory/VectorMeasure/Variation/Defs.lean,Mathlib/MeasureTheory/VectorMeasure/Variation/Lemmas.lean |
6 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
16-101 16 days ago |
16-102 16 days ago |
0-0 0 seconds |
| 30312 |
kckennylau author:kckennylau |
feat(RingTheory): define graded ring homomorphisms |
This PR defines graded ring homomorphisms, which are ring homomorphisms that preserve the grading. We also provide the basic properties (aka the "API").
Zulip discussion: [#mathlib4 > Graded Ring Hom](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Graded.20Ring.20Hom/with/543601500)
---
Split from #26061.
- [ ] depends on: #30355
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
merge-conflict
blocked-by-other-PR
|
360/0 |
Mathlib.lean,Mathlib/Data/FunLike/GradedFunLike.lean,Mathlib/RingTheory/GradedAlgebra/RingHom.lean |
3 |
7 |
['github-actions', 'kckennylau', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'plp127'] |
nobody |
16-94 16 days ago |
16-95 16 days ago |
1-46922 1 day |
| 30334 |
kckennylau author:kckennylau |
feat(RingTheory): define maps of homogeneous ideals |
In this file we define `HomogeneousIdeal.map` and `HomogeneousIdeal.comap`, similar to and based on the existing `Ideal.map` and `Ideal.comap`. More concretely, a graded ring homomorphism `𝒜 →+*ᵍ ℬ` induces a "Galois connection" between the homogeneous ideals in `𝒜` and the homogeneous ideals in `ℬ`.
---
Split from #26061.
- [ ] depends on: #30312
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
merge-conflict
blocked-by-other-PR
|
441/0 |
Mathlib.lean,Mathlib/RingTheory/GradedAlgebra/Hom.lean,Mathlib/RingTheory/GradedAlgebra/Homogeneous/Ideal.lean,Mathlib/RingTheory/GradedAlgebra/Homogeneous/Maps.lean |
4 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
16-90 16 days ago |
16-91 16 days ago |
0-1744 29 minutes |
| 30365 |
kckennylau author:kckennylau |
feat(RingTheory): define R-linear graded algebra homomorphism |
This PR defines R-linear graded algebra homomorphisms, which are R-algebra homomorphisms that preserve the grading. We also provide the basic properties (aka the "API").
Zulip discussion: [#mathlib4 > redefine Graded Algebra](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/redefine.20Graded.20Algebra/near/543847326)
---
Split from #26061.
- [ ] depends on: #30355
- [ ] depends on: #30312
[](https://gitpod.io/from-referrer/)
|
merge-conflict
blocked-by-other-PR
|
642/0 |
Mathlib.lean,Mathlib/Data/FunLike/GradedFunLike.lean,Mathlib/RingTheory/GradedAlgebra/AlgHom.lean,Mathlib/RingTheory/GradedAlgebra/RingHom.lean |
4 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
16-78 16 days ago |
16-79 16 days ago |
0-578 9 minutes |
| 30367 |
kckennylau author:kckennylau |
feat(Data): define grading-preserving isomorphisms |
The class `GradedEquivLike E 𝒜 ℬ` says that `E` is a type of grading-preserving isomorphisms between `𝒜` and `ℬ`. It is the combination of `GradedFunLike E 𝒜 ℬ` and `EquivLike E A B`.
---
- [ ] depends on: #30355
[](https://gitpod.io/from-referrer/)
|
t-data
merge-conflict
blocked-by-other-PR
|
78/0 |
Mathlib.lean,Mathlib/Data/FunLike/Graded.lean |
2 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
16-77 16 days ago |
16-78 16 days ago |
0-3399 56 minutes |
| 30374 |
FLDutchmann author:FLDutchmann |
feat(Tactic): `algebra` and `polynomial` tactic suite |
Implement a suite of tactics for normalizing expressions in an algebra over a ring. Handles all of the normal `ring` operations as well as scalar multiplication over a fixed base ring. Using these, implement tactics to normalize `(Mv)Polynomial` expressions into a sum-of-monomials form.
Specifically,
* `algebra` proves equality of expressions in an algebra over a ring like `ring1`
* `algebra_nf` puts expressions in an algebra into a normal form, like `ring_nf`
* `match_scalars_alg` (name pending) closes an equality goal by calling `algebra_nf` and creating side goals equating matching coefficients in the base ring. Like `match_scalars`.
* `polynomial` proves equality of (mv)polynomials
* `polynomial_nf` expands polynomials into a sum-of-monomials form, combining coefficients in the base ring (e.g. `C a * X + C b * X` normalizes to `C(a+b) * X`
* `match_coefficients` expands polynomials and produces side goals equating matching coefficients.
- [ ] depends on: #31506
- [ ] depends on: #31508
- [ ] depends on: #31513
---
[](https://gitpod.io/from-referrer/)
|
t-meta
merge-conflict
awaiting-author
blocked-by-other-PR
|
2371/0 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Algebra.lean,Mathlib/Tactic/Algebra/Lemmas.lean,Mathlib/Tactic/Polynomial.lean,Mathlib/Tactic/Polynomial/Core.lean,MathlibTest/Polynomial.lean,MathlibTest/algebra.lean,scripts/noshake.json |
9 |
7 |
['FLDutchmann', 'github-actions', 'hrmacbeth', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
16-74 16 days ago |
16-75 16 days ago |
0-0 0 seconds |
| 30379 |
kckennylau author:kckennylau |
feat(RingTheory): isomorphism of graded rings |
We define `GradedRingEquiv 𝒜 ℬ` to mean isomorphisms of graded rings, with notation `𝒜 ≃+*ᵍ ℬ`. When possible, instead of parametrizing results over `(e : 𝒜 ≃+*ᵍ ℬ)`, you should parametrize over `[GradedEquivLike E 𝒜 ℬ] [RingEquivClass E A B] (e : E)`.
Zulip discussion: [How to define graded ring isomorphisms?](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/How.20to.20define.20graded.20ring.20isomorphisms.3F/with/543962394)
---
Split from #26061.
- [ ] depends on: #30355
- [ ] depends on: #30312
- [ ] depends on: #30367
[](https://gitpod.io/from-referrer/)
|
merge-conflict
blocked-by-other-PR
|
825/0 |
Mathlib.lean,Mathlib/Data/FunLike/Graded.lean,Mathlib/RingTheory/GradedAlgebra/RingEquiv.lean,Mathlib/RingTheory/GradedAlgebra/RingHom.lean |
4 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
16-72 16 days ago |
16-72 16 days ago |
0-3140 52 minutes |
| 30985 |
erdOne author:erdOne |
feat(AlgbraicGeometry), `Hom(-, X)` commutes with inverse limits for schemes of finite presentation |
---
- [ ] depends on: #30988
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebraic-geometry
merge-conflict
blocked-by-other-PR
|
523/28 |
Mathlib/AlgebraicGeometry/AffineTransitionLimit.lean |
1 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
15-86151 15 days ago |
15-86152 15 days ago |
0-4846 1 hour |
| 31083 |
joelriou author:joelriou |
feat(CategoryTheory): properties of objects for pseudofunctors to Cat |
Given `F : Pseudofunctor B Cat`, we introduce a type `F.ObjectProperty` which consists of properties `P` of objects for all categories `F.obj X` for `X : B`. The typeclass `P.IsClosedUnderMapObj` expresses that this property is preserved by the application of the functors `F.map`: this allows to define a sub-pseudofunctor `P.fullsubcategory : Pseudofunctor B Cat`.
---
- [ ] depends on: #26446.
[](https://gitpod.io/from-referrer/)
|
t-category-theory
merge-conflict
blocked-by-other-PR
WIP
|
140/0 |
Mathlib.lean,Mathlib/CategoryTheory/Bicategory/Functor/Cat/ObjectProperty.lean |
2 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
15-86129 15 days ago |
15-86130 15 days ago |
0-1 1 second |
| 31580 |
grunweg author:grunweg |
feat: towards `ContMDiff` support in fun_prop |
Create a `find_model` tactic for solving `ModelWithCorners k E H` goals,
and a #find_model command to simplify testing it. (Both implementations are a bit hacky right now.)
next step: extend the tactic, test that it works well
then try to hook it up to fun_prop
---
- [ ] depends on: #30463
[](https://gitpod.io/from-referrer/)
|
t-differential-geometry
t-meta
merge-conflict
blocked-by-other-PR
WIP
|
1254/64 |
Mathlib/Geometry/Manifold/Instances/UnitsOfNormedAlgebra.lean,Mathlib/Geometry/Manifold/Notation.lean,Mathlib/Geometry/Manifold/TestFunPropM.lean,MathlibTest/DifferentialGeometry/Notation.lean,MathlibTest/DifferentialGeometry/NotationAdvanced.lean,mathlib-immersions |
6 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
15-81400 15 days ago |
15-81401 15 days ago |
0-1 1 second |
| 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$ |
194/3 |
Mathlib.lean,Mathlib/Geometry/Group/Marking.lean,Mathlib/Topology/Algebra/ConstMulAction.lean,Mathlib/Topology/Algebra/Group/Quotient.lean |
4 |
15 |
['YaelDillies', 'b-mehta', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
15-75255 15 days ago |
15-75273 15 days ago |
22-16818 22 days |
| 30339 |
grunweg author:grunweg |
feat: extend a tangent vector for a locally smooth vector field |
Given a vector bundle `V` over `M` and a vector `X` in the fibre `E x` some point `x`,
construct a section of `V` which is smooth near `x` and has value `X` at `x`.
This will be used to prove the tensoriality of covariant derivatives.
From the path towards geodesics and the Levi-Civita connection.
Co-authored-by: Patrick Massot [patrickmassot@free.fr](mailto:patrickmassot@free.fr)
---
TODO: order of variables --- first e then b, or the other way around?
should the new definition be namespaced, e.g. in the Trivialization namespace?
- [ ] depends on: #30083
[](https://gitpod.io/from-referrer/)
|
t-differential-geometry
merge-conflict
blocked-by-other-PR
|
435/14 |
Mathlib/Geometry/Manifold/VectorBundle/LocalFrame.lean |
1 |
4 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
15-67425 15 days ago |
15-67426 15 days ago |
0-850 14 minutes |
| 31338 |
grunweg author:grunweg |
chore: move Pretrivialization, Trivialization to the Bundle namespace |
As suggested in #30083.
---
- [ ] depends on: #30083
[](https://gitpod.io/from-referrer/)
|
t-differential-geometry
merge-conflict
blocked-by-other-PR
|
400/71 |
Mathlib/Geometry/Manifold/MFDeriv/UniqueDifferential.lean,Mathlib/Geometry/Manifold/VectorBundle/Basic.lean,Mathlib/Geometry/Manifold/VectorBundle/LocalFrame.lean,Mathlib/Geometry/Manifold/VectorBundle/MDifferentiable.lean,Mathlib/Topology/FiberBundle/Constructions.lean,Mathlib/Topology/FiberBundle/Trivialization.lean,Mathlib/Topology/VectorBundle/Basic.lean,Mathlib/Topology/VectorBundle/Constructions.lean,Mathlib/Topology/VectorBundle/Hom.lean |
9 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
15-62877 15 days ago |
15-62878 15 days ago |
0-2491 41 minutes |
| 31339 |
grunweg author:grunweg |
Movelemma |
---
- [ ] depends on: #31338
[](https://gitpod.io/from-referrer/)
|
merge-conflict
blocked-by-other-PR
|
415/78 |
Mathlib/Geometry/Manifold/MFDeriv/UniqueDifferential.lean,Mathlib/Geometry/Manifold/VectorBundle/Basic.lean,Mathlib/Geometry/Manifold/VectorBundle/LocalFrame.lean,Mathlib/Geometry/Manifold/VectorBundle/MDifferentiable.lean,Mathlib/Topology/FiberBundle/Constructions.lean,Mathlib/Topology/FiberBundle/Trivialization.lean,Mathlib/Topology/VectorBundle/Basic.lean,Mathlib/Topology/VectorBundle/Constructions.lean,Mathlib/Topology/VectorBundle/Hom.lean |
9 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
15-62875 15 days ago |
15-62877 15 days ago |
0-1962 32 minutes |
| 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 |
15-60477 15 days ago |
445-11976 1 year ago |
1-72084 1 day |
| 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 |
15-60371 15 days ago |
unknown |
unknown |
| 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 |
15-60356 15 days ago |
390-77741 1 year ago |
0-1869 31 minutes |
| 19607 |
madvorak author:madvorak |
feat: block matrices are 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 |
15-60341 15 days ago |
133-81075 4 months ago |
0-0 0 seconds |
| 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
merge-conflict
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 |
4 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
15-60080 15 days ago |
71-22715 2 months 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
merge-conflict
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 |
4 |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
15-60060 15 days ago |
71-22716 2 months ago |
0-850 14 minutes |
| 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
merge-conflict
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 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
15-60000 15 days ago |
16-1559 16 days ago |
15-65390 15 days |
| 29792 |
robertmaxton42 author:robertmaxton42 |
feat(RelCWComplex): a (relative, concrete) CW complex is the colimit of its skeleta |
Adds:
* `RelCWComplex.Subcomplex.isCoherentWith_cover`: a (relative) CW complex is coherent with any collection of subcomplexes that cover.
* `RelCWComplex.descBySkeletonLT` and `descBySkeleton`: construct a continuous map from a complex by providing a family of compatible maps from each skeleton and the base. `CWComplex.descBySkeleton` skips the base.
- [ ] depends on: #29788
- [ ] depends on: #29790
---
[](https://gitpod.io/from-referrer/)
|
large-import
merge-conflict
blocked-by-other-PR
|
672/31 |
Mathlib/Data/Set/Subset.lean,Mathlib/Data/Set/UnionLift.lean,Mathlib/Topology/CWComplex/Classical/Basic.lean,Mathlib/Topology/CWComplex/Classical/Finite.lean,Mathlib/Topology/CWComplex/Classical/Subcomplex.lean,Mathlib/Topology/Category/TopCat/Limits/Products.lean,Mathlib/Topology/Coherent.lean,Mathlib/Topology/Constructions.lean,Mathlib/Topology/Constructions/SumProd.lean,Mathlib/Topology/ContinuousMap/Basic.lean |
10 |
4 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'scholzhannah'] |
nobody |
15-59643 15 days ago |
16-279 16 days ago |
0-1375 22 minutes |
| 29790 |
robertmaxton42 author:robertmaxton42 |
feat(IsCoherentWith) : families of maps from a coherent collection of subspaces lift uniquely to maps from the total space |
* Adds `IsCoherentWith.liftCover`, which lifts a compatible family of continuous maps from each member of a coherent set of subspaces to a single continuous map on the whole space.
* Adds `IsCoherentWith.liftCover'`, which does the same but for a set of coherent subspaces given as the range of a function into `Set X` rather than as an explicit `Set (Set X).`
- [ ] depends on: #29788
---
[](https://gitpod.io/from-referrer/)
|
large-import
merge-conflict
blocked-by-other-PR
|
350/3 |
Mathlib/Data/Set/Subset.lean,Mathlib/Data/Set/UnionLift.lean,Mathlib/Topology/Category/TopCat/Limits/Products.lean,Mathlib/Topology/Coherent.lean,Mathlib/Topology/Constructions.lean,Mathlib/Topology/Constructions/SumProd.lean,Mathlib/Topology/ContinuousMap/Basic.lean |
7 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
15-59638 15 days ago |
16-281 16 days ago |
0-4627 1 hour |
| 28718 |
imbrem author:imbrem |
feat: class for 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.
- [ ] depends on: #30150 |
new-contributor
t-category-theory
merge-conflict
awaiting-author
blocked-by-other-PR
|
290/0 |
Mathlib.lean,Mathlib/CategoryTheory/ChosenFiniteCoproducts.lean |
2 |
9 |
['YaelDillies', 'github-actions', 'imbrem', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'robin-carlier'] |
nobody |
15-59621 15 days ago |
16-1036 16 days ago |
0-24930 6 hours |
| 30352 |
kckennylau author:kckennylau |
feat(RingTheory): Homogeneous localization of tensor product |
Let `𝒜` be a graded `R`-algebra, and `S` be an `R`-algebra. Then `S ⊗[R] 𝒜` is a graded
`S`-algebra with the same grading.
Let `W` be a homogeneous submonoid of `𝒜`. Then `(S⊗[R]𝒜)[(1⊗W)⁻¹]₀ ≅ S ⊗[R] (𝒜[W⁻¹]₀)`.
---
Split from #26061.
- [x] depends on: #30173
- [ ] depends on: #30322
[](https://gitpod.io/from-referrer/)
|
merge-conflict
blocked-by-other-PR
WIP
|
563/48 |
Mathlib.lean,Mathlib/Algebra/DirectSum/Basic.lean,Mathlib/Algebra/DirectSum/Decomposition.lean,Mathlib/Algebra/DirectSum/Module.lean,Mathlib/Algebra/Order/Module/HahnEmbedding.lean,Mathlib/LinearAlgebra/DirectSum/Finsupp.lean,Mathlib/LinearAlgebra/DirectSum/TensorProduct.lean,Mathlib/LinearAlgebra/TensorProduct/Decomposition.lean,Mathlib/LinearAlgebra/TensorProduct/Tower.lean,Mathlib/RingTheory/Flat/Basic.lean,Mathlib/RingTheory/Flat/FaithfullyFlat/Basic.lean,Mathlib/RingTheory/GradedAlgebra/TensorLocalization.lean,Mathlib/RingTheory/GradedAlgebra/TensorProduct.lean |
13 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
15-59600 15 days ago |
35-65665 1 month ago |
0-9 9 seconds |
| 31411 |
CoolRmal author:CoolRmal |
feat: a convex lower-semicontinuous function is the supremum of a sequence of affine functions in a separable space |
This lemma is needed in the proof of conditional Jensen's inequality: #27953
The lemmas in this PR need the RCLike API, so it is not suitable to put them in Mathlib.Topology.Semicontinuous or Mathlib.Analysis.Convex.Function as they does not import RCLike. I tried to put these lemmas in a RCLike related file but I encountered warnings about import (e.g. Modules starting with Mathlib.Topology are not allowed to import modules starting with ...). Therefore, I temporarily put them in [Mathlib/MeasureTheory/Function/ConditionalExpectation/CondJensen.lean](https://github.com/leanprover-community/mathlib4/pull/31411/files#diff-930cc0818908e1ab51f74f3729ae6de8ed43f7914e94ca07c619f48a4c49aa9c).
---
- [ ] depends on: #31180
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-analysis
merge-conflict
blocked-by-other-PR
|
337/10 |
Mathlib.lean,Mathlib/Analysis/LocallyConvex/Separation.lean,Mathlib/MeasureTheory/Function/ConditionalExpectation/Basic.lean,Mathlib/MeasureTheory/Function/ConditionalExpectation/CondJensen.lean |
4 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
15-59559 15 days ago |
15-81683 15 days ago |
0-129 2 minutes |
| 31134 |
thorimur author:thorimur |
chore: use `whenLinterActivated` in linters |
Replaces boilerplate in linters with `whenLinterActivated` or `whenLinterOption` where possible.
---
- [ ] depends on: #31133
[](https://gitpod.io/from-referrer/)
|
blocked-by-other-PR |
221/189 |
Mathlib.lean,Mathlib/Lean/Linter.lean,Mathlib/Tactic/Linter/CommandRanges.lean,Mathlib/Tactic/Linter/CommandStart.lean,Mathlib/Tactic/Linter/DeprecatedModule.lean,Mathlib/Tactic/Linter/DocPrime.lean,Mathlib/Tactic/Linter/FlexibleLinter.lean,Mathlib/Tactic/Linter/GlobalAttributeIn.lean,Mathlib/Tactic/Linter/HashCommandLinter.lean,Mathlib/Tactic/Linter/Header.lean,Mathlib/Tactic/Linter/Lint.lean,Mathlib/Tactic/Linter/MinImports.lean,Mathlib/Tactic/Linter/Multigoal.lean,Mathlib/Tactic/Linter/OldObtain.lean,Mathlib/Tactic/Linter/PPRoundtrip.lean,Mathlib/Tactic/Linter/Style.lean,Mathlib/Tactic/Linter/UnusedTactic.lean,Mathlib/Tactic/Linter/UpstreamableDecl.lean,Mathlib/Util/CountHeartbeats.lean,scripts/lint-style.lean |
20 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
15-21225 15 days ago |
15-21981 15 days ago |
0-0 0 seconds |
| 31513 |
FLDutchmann author:FLDutchmann |
feat(Tactic): `polynomial` tactic |
Implement tactic for proving equality of polynomials.
This tactic is part of a larger suite (see https://github.com/leanprover-community/mathlib4/pull/30374).
- [ ] depends on: #31508
---
[](https://gitpod.io/from-referrer/)
|
t-meta
merge-conflict
blocked-by-other-PR
|
1824/6 |
Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Algebra/Basic.lean,Mathlib/Tactic/Algebra/Lemmas.lean,Mathlib/Tactic/Polynomial/Basic.lean,Mathlib/Tactic/Polynomial/Core.lean,Mathlib/Util/Qq.lean,MathlibTest/Algebra.lean,MathlibTest/Polynomial.lean,scripts/noshake.json |
10 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
Vierkantor assignee:Vierkantor |
14-49164 14 days ago |
15-81661 15 days ago |
0-1388 23 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
- [x] depends on: #27021
Baby version of #27025.
[](https://gitpod.io/from-referrer/)
|
t-differential-geometry
merge-conflict
blocked-by-other-PR
|
390/11 |
Mathlib.lean,Mathlib/Analysis/InnerProductSpace/GramSchmidtOrtho.lean,Mathlib/Geometry/Manifold/VectorBundle/GramSchmidtOrtho.lean,scripts/noshake.json |
4 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
13-38706 13 days ago |
18-63076 18 days ago |
0-696 11 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.
- [x] depends on: #27021
- [x] depends on: #27023
- [ ] depends on: #27024
[](https://gitpod.io/from-referrer/)
|
t-differential-geometry
merge-conflict
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 |
6 |
['faenuccio', 'github-actions', 'grunweg', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
13-38702 13 days ago |
18-63200 18 days ago |
0-316 5 minutes |
| 29777 |
yuanyi-350 author:yuanyi-350 |
feat(Functional Analysis): closed Range Theorem |
- [ ] depends on: #29151 [Corollary of Hahn-Banach theorem]
- [ ] depends on: #29776 [refactor ContinuousLinearMap.isOpenMap by separating it into sublemmas]
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-analysis
awaiting-author
blocked-by-other-PR
WIP
|
237/25 |
Mathlib/Analysis/LocallyConvex/Separation.lean,Mathlib/Analysis/Normed/Operator/Banach.lean,Mathlib/Analysis/Normed/Operator/ClosedRange.lean,Mathlib/Analysis/RCLike/Lemmas.lean,Mathlib/Topology/Order/OrderClosed.lean |
5 |
4 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
faenuccio assignee:faenuccio |
12-81728 12 days ago |
12-81896 12 days ago |
0-634 10 minutes |
| 30982 |
jsm28 author:jsm28 |
feat(Geometry/Euclidean/Angle/Incenter): angle bisection and the incenter |
Add lemmas relating the incenter and excenters of a simplex to angle bisection, both generally for a simplex and more specifically with oriented angles for a triangle.
More specific lemmas for a simplex (identifying exactly which excenter corresponds to which bisectors) will require various additional API for bisectors of angles betweeen oriented affine subspaces (but for the most common applications to typical plane geometry problems, I expect the triangle lemmas with oriented angles to be more useful).
---
- [ ] depends on: #30474
- [ ] depends on: #30477
- [ ] depends on: #30600
- [ ] depends on: #30703
- [ ] depends on: #30938
- [ ] depends on: #30981
[](https://gitpod.io/from-referrer/)
|
t-euclidean-geometry
blocked-by-other-PR
|
424/4 |
Mathlib.lean,Mathlib/Geometry/Euclidean/Angle/Bisector.lean,Mathlib/Geometry/Euclidean/Angle/Incenter.lean |
3 |
4 |
['github-actions', 'jsm28', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
12-29815 12 days ago |
15-76876 15 days ago |
0-2478 41 minutes |
| 31670 |
edwin1729 author:edwin1729 |
feat(Topology/Order): Scott Topology is Sober over Algebraic DCPO |
---
[Zulip discussion](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/.3E.20Algebraic.20complete.20partial.20order.20and.20domain.20theory/with/536359313) here
(2/2) PR to prove result in Stone Duality. Here we prove that Scott Topologies over Algebraic DCPOs are sober.
- [ ] depends on: #31662
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-topology
blocked-by-other-PR
|
523/0 |
Mathlib.lean,Mathlib/Topology/Order/ScottTopologyDCPO.lean,docs/references.bib |
3 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
11-42838 11 days ago |
11-42858 11 days ago |
0-0 0 seconds |
| 30831 |
chrisflav author:chrisflav |
feat(AlgebraicGeometry): the fpqc topology |
We define the fpqc topology on the category of schemes as the intersection of the quasi-compact topology with the flat topology.
From Proetale.
---
- [x] depends on: #30835
- [x] depends on: #30906
- [x] depends on: #30910
- [ ] depends on: #32042
[](https://gitpod.io/from-referrer/)
|
t-algebraic-geometry
blocked-by-other-PR
|
407/1 |
Mathlib.lean,Mathlib/AlgebraicGeometry/Cover/QuasiCompact.lean,Mathlib/AlgebraicGeometry/Morphisms/Affine.lean,Mathlib/AlgebraicGeometry/Morphisms/QuasiCompact.lean,Mathlib/AlgebraicGeometry/Morphisms/UnderlyingMap.lean,Mathlib/AlgebraicGeometry/Sites/MorphismProperty.lean,Mathlib/AlgebraicGeometry/Sites/QuasiCompact.lean,Mathlib/Topology/Sets/CompactOpenCovered.lean,Mathlib/Topology/Spectral/Prespectral.lean |
9 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
10-78605 10 days ago |
10-78606 10 days ago |
0-1076 17 minutes |
| 29764 |
ScottCarnahan author:ScottCarnahan |
feat(Algebra/Vertex): API up to residue products (WIP) |
This PR contains definitions leading up to the residue product of vertex operators and some basic properties.
Parts will be split off as smaller PRs when I have time.
---
- [ ] depends on: #25831
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
blocked-by-other-PR
label:t-algebra$ |
1159/27 |
Mathlib.lean,Mathlib/Algebra/Vertex/HVertexOperator.lean,Mathlib/Algebra/Vertex/VertexOperator.lean,Mathlib/RingTheory/Binomial.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/Summable.lean |
10 |
4 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
10-47458 10 days ago |
10-47459 10 days ago |
0-25208 7 hours |
| 28248 |
YaelDillies author:YaelDillies |
feat: binomial random variables |
Define the binomial distribution and compute the expectation, variance, conditional variance of a binomial random variable.
From MiscYD
---
- [ ] depends on: #31908
- [x] depends on: #31910
- [x] depends on: #31942
- [x] depends on: #31947
[](https://gitpod.io/from-referrer/)
|
t-measure-probability
blocked-by-other-PR
|
397/4 |
Mathlib.lean,Mathlib/MeasureTheory/Integral/Bochner/Set.lean,Mathlib/MeasureTheory/Measure/Dirac.lean,Mathlib/MeasureTheory/Measure/Restrict.lean,Mathlib/Probability/Distributions/Bernoulli.lean,Mathlib/Probability/Distributions/Binomial.lean,Mathlib/Probability/HasLaw.lean,Mathlib/Probability/Moments/Variance.lean |
8 |
52 |
['DavidLedvinka', 'RemyDegenne', 'YaelDillies', 'github-actions', 'kex-y', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'pfaffelh', 'themathqueen'] |
kex-y assignee:kex-y |
9-84990 9 days ago |
12-44667 12 days ago |
28-39091 28 days |
| 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
- uniqueness of the Levi-Civita connection
- Christoffel symbols
- in progress: existence of the Levi-Civita connection (connection done; torsion-freeness and compatibility in progress)
- custom elaborators for sections in a vector bundle (converting dependent to non-dependent functions)
- custom elaborators for inferring a model with corners, in differentiability/smoothness definitions
- a `#check'` command and tactic which only shows explicit arguments
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
- [x] depends on: #26870
- [x] 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
- [x] depends on: #27021
- [x] depends on: #30307
- [x] depends on: #27023
- [ ] depends on: #27024
- [ ] depends on: #27025
- [x] depends on: #30338
- [ ] depends on: #30083
- [ ] depends on: #30339
- [ ] depends on: #31194
[](https://gitpod.io/from-referrer/)
|
t-differential-geometry
merge-conflict
blocked-by-other-PR
|
5100/305 |
Mathlib.lean,Mathlib/Geometry/Manifold/CheatSheet.md,Mathlib/Geometry/Manifold/PartitionOfUnity.lean,Mathlib/Geometry/Manifold/Riemannian/ExistsRiemannianMetric.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 |
17 |
n/a |
['github-actions', 'grunweg', 'idontgetoutmuch', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
9-16141 9 days ago |
unknown |
unknown |
| 31873 |
wwylele author:wwylele |
refactor: re-prove Euler's partition theorem from Glaisher's theorem |
Less code to maintain is good. I hope the authors of the original proof are fine with this...
---
- [ ] depends on: #30618
[](https://gitpod.io/from-referrer/)
|
file-removed
merge-conflict
blocked-by-other-PR
|
214/395 |
Archive.lean,Archive/Wiedijk100Theorems/Partition.lean,Mathlib.lean,Mathlib/Combinatorics/Enumerative/Partition/Basic.lean,Mathlib/Combinatorics/Enumerative/Partition/GenFun.lean,Mathlib/Combinatorics/Enumerative/Partition/Glaisher.lean,Mathlib/RingTheory/PowerSeries/PiTopology.lean,docs/100.yaml,docs/1000.yaml |
9 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
9-11595 9 days ago |
9-11596 9 days ago |
0-610 10 minutes |
| 30463 |
grunweg author:grunweg |
feat: support products and disjoint unions in the differential geometry elaborators |
Add support for inferring a model with corners on
- products of manifolds
- disjoint unions of manifolds
- an open subset of a manifold
Note that these can be nested (e.g., a product with multiple factors, a disjoint union of four manifolds or combinations of these).
For binary products of normed spaces, we intentionally refuse to infer a model with corners, as there are two different possible options which are propositionally, but not definitionally equal. For now, we emit a warning to this effect instead. A future PR may remove it (and infer one of these variants): see [zulip discussion](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Differential.20geometry.20elaborators.20experiment/near/544942546).
---
~~Baby version of #30421.~~ This seems to be the full version. Open subsets do not work well yet, that's a bug to fix.
- [ ] depends on: #30744
- [ ] depends on: #30879
[](https://gitpod.io/from-referrer/)
|
t-differential-geometry
t-meta
merge-conflict
blocked-by-other-PR
|
905/63 |
Mathlib/Geometry/Manifold/Instances/UnitsOfNormedAlgebra.lean,Mathlib/Geometry/Manifold/Notation.lean,MathlibTest/DifferentialGeometry/Notation.lean,MathlibTest/DifferentialGeometry/NotationAdvanced.lean,mathlib-immersions |
5 |
6 |
['github-actions', 'grunweg', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
thorimur assignee:thorimur |
8-77013 8 days ago |
16-67 16 days ago |
0-484 8 minutes |
| 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).
---
- [ ] depends on: #32134
[](https://gitpod.io/from-referrer/)
|
t-combinatorics
blocked-by-other-PR
|
139/22 |
Mathlib/Algebra/Order/Monoid/Canonical/Basic.lean,Mathlib/Combinatorics/SimpleGraph/Extremal/TuranDensity.lean,Mathlib/Topology/Instances/NNReal/Lemmas.lean |
3 |
22 |
['YaelDillies', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'mitchell-horner'] |
YaelDillies assignee:YaelDillies |
8-72381 8 days ago |
8-72382 8 days ago |
69-44187 69 days |
| 31113 |
515801431 author:515801431 |
feat(Mathlib/Combinatorics/Enumerative/Polya.lean): Add additional theorem in `Polya.lean` |
---
- [ ] depends on: #30525
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
t-combinatorics
blocked-by-other-PR
|
302/0 |
Mathlib.lean,Mathlib/Combinatorics/Enumerative/Polya.lean |
2 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
b-mehta assignee:b-mehta |
8-68916 8 days ago |
8-69629 8 days ago |
22-58765 22 days |
| 30881 |
FlAmmmmING author:FlAmmmmING |
feat(RingTheory/PowerSeries/Schroder.lean): Define the generating function for large and small Schroder number |
Define the generating function for large and small Schroder number.
Main result : Prove some lemmas and the generating function of large Schroder.
Todo : Prove the generating function of small Schroder.
---
- [ ] depends on: #30609
---
[](https://gitpod.io/from-referrer/)
|
new-contributor
blocked-by-other-PR
|
352/1 |
Mathlib.lean,Mathlib/Combinatorics/Enumerative/Catalan.lean,Mathlib/RingTheory/PowerSeries/Schroder.lean |
3 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
dwrensha assignee:dwrensha |
8-68894 8 days ago |
8-70424 8 days ago |
31-71873 31 days |
| 31332 |
sinhp author:sinhp |
feat(CategoryTheory): Exponentiable morphisms |
We define an exponentiable morphism `f : I ⟶ J` to be a morphism with a chosen pullback functor
`Over J ⥤ Over I` together with a right adjoint, called the pushforward functor.
We use this PR in the PR branch `lccc-basic`.
```mermaid
graph TD
A[ChosenPullbacksAlong.lean] --> A'[Over.lean]
A' --> B[Sections.lean]
A --> C[ExponentiableMorphism.lean]
B --> D[Basic.lean]
C --> D
D --> E[Types.lean]
E --> F[Presheaves.lean]
D --> G[Beck-Chevalley.lean]
%% Define highlight style
classDef highlight fill:#ffe599,stroke:#d4a017,stroke-width:2px;
%% Apply to one node
class C highlight;
```
---
- [x] depends on: #31033
- [ ] depends on: #31433
[](https://gitpod.io/from-referrer/)
|
t-category-theory
blocked-by-other-PR
|
167/0 |
Mathlib.lean,Mathlib/CategoryTheory/LocallyCartesianClosed/ExponentiableMorphism.lean |
2 |
6 |
['github-actions', 'joelriou', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'sinhp'] |
nobody |
8-57458 8 days ago |
8-73417 8 days ago |
0-14 14 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-55958 8 days ago |
90-77952 2 months ago |
0-0 0 seconds |
| 31729 |
thorimur author:thorimur |
chore: log on theorem type signature in unused instances in type linters |
Logs on the type signature in the unused instances in types linter, and tests this using `#guard_msgs (positions := true)`.
---
- [ ] depends on: #31730
- [x] depends on: #31142
[](https://gitpod.io/from-referrer/)
|
large-import
merge-conflict
blocked-by-other-PR
|
636/3 |
Mathlib.lean,Mathlib/Lean/Elab/InfoTree.lean,Mathlib/Lean/Environment.lean,Mathlib/Lean/Expr.lean,Mathlib/Lean/Expr/Basic.lean,Mathlib/Lean/Syntax.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter.lean,Mathlib/Tactic/Linter/DirectoryDependency.lean,Mathlib/Tactic/Linter/UnusedInstancesInType.lean,Mathlib/Util/DeclarationManipulation.lean,MathlibTest/UnusedInstancesInType.lean |
12 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
8-40788 8 days ago |
15-81362 15 days ago |
0-697 11 minutes |
| 32157 |
peabrainiac author:peabrainiac |
feat(Analysis/Calculus): Hadamard's lemma |
Add [Hadamard's lemma](https://en.wikipedia.org/wiki/Hadamard%27s_lemma) for functions from finite-dimensional normed spaces to Banach spaces.
---
- [ ] depends on: #31141
[](https://gitpod.io/from-referrer/)
|
t-analysis
blocked-by-other-PR
|
314/5 |
Mathlib.lean,Mathlib/Analysis/Calculus/Hadamard.lean,Mathlib/Analysis/Calculus/ParametricIntegral.lean,Mathlib/Analysis/Calculus/ParametricIntervalIntegral.lean,Mathlib/MeasureTheory/Integral/DominatedConvergence.lean |
5 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
8-31323 8 days ago |
8-31324 8 days ago |
0-1385 23 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).
- [ ] depends on: #30001
- [ ] depends on: #29995
[](https://gitpod.io/from-referrer/)
|
t-order
merge-conflict
awaiting-author
blocked-by-other-PR
|
500/104 |
Mathlib.lean,Mathlib/Order/Completion.lean,Mathlib/Order/Concept.lean |
3 |
23 |
['YaelDillies', 'github-actions', 'leanprover-community-bot-assistant', 'linesthatinterlace', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'vihdzp'] |
nobody |
8-1468 8 days ago |
16-1355 16 days ago |
0-19769 5 hours |
| 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 |
t-order
awaiting-CI
blocked-by-other-PR
WIP
|
12/0 |
Mathlib/Algebra/Order/GroupWithZero/Unbundled/Basic.lean |
1 |
47 |
['Vierkantor', 'YaelDillies', 'faenuccio', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
7-86184 7 days ago |
7-86192 7 days ago |
5-22106 5 days |
| 31018 |
joelriou author:joelriou |
feat(CategoryTheory): the κ-accessible category of κ-directed posets |
WIP
---
- [ ] depends on: #30727
- [ ] depends on: #31767
- [x] depends on: #29519
- [x] depends on: #29543
- [x] depends on: #29565
- [x] depends on: #29854
- [x] depends on: #30459
- [ ] depends on: #30605
- [ ] depends on: #31426
- [ ] depends on: #31421
- [x] depends on: #30633
- [x] depends on: #30634
- [x] depends on: #30693
- [x] depends on: #30696
- [x] depends on: #30781
[](https://gitpod.io/from-referrer/)
|
t-category-theory
merge-conflict
blocked-by-other-PR
WIP
|
1231/5 |
Mathlib.lean,Mathlib/CategoryTheory/Comma/Arrow.lean,Mathlib/CategoryTheory/MorphismProperty/Basic.lean,Mathlib/CategoryTheory/MorphismProperty/HasCardinalLT.lean,Mathlib/CategoryTheory/ObjectProperty/HasCardinalLT.lean,Mathlib/CategoryTheory/ObjectProperty/LimitsClosure.lean,Mathlib/CategoryTheory/Presentable/Basic.lean,Mathlib/CategoryTheory/Presentable/CardinalDirectedPoset.lean,Mathlib/CategoryTheory/Presentable/CardinalFilteredPresentation.lean,Mathlib/CategoryTheory/Presentable/Directed.lean,Mathlib/CategoryTheory/Presentable/IsCardinalFiltered.lean,Mathlib/CategoryTheory/Presentable/SharplyLT.lean,Mathlib/CategoryTheory/Presentable/Type.lean,Mathlib/Order/Category/PartOrdEmb.lean,docs/references.bib |
15 |
n/a |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
7-83421 7 days ago |
unknown |
unknown |
| 31805 |
joelriou author:joelriou |
feat(AlgebraicTopology): horns in Δ[n] as multicoequalizers |
Some API is also introduced for the particular case of inner horns in `Δ[3]`.
Co-authored-by: Nick Ward gio256@protonmail.com
From https://github.com/joelriou/topcat-model-category
---
- [ ] depends on: #31802
- [x] depends on: #31797
[](https://gitpod.io/from-referrer/)
|
t-algebraic-topology
blocked-by-other-PR
WIP
|
424/0 |
Mathlib.lean,Mathlib/AlgebraicTopology/SimplicialSet/Horn.lean,Mathlib/AlgebraicTopology/SimplicialSet/HornColimits.lean,Mathlib/AlgebraicTopology/SimplicialSet/StdSimplex.lean,Mathlib/AlgebraicTopology/SimplicialSet/Subcomplex.lean,Mathlib/CategoryTheory/Limits/Shapes/Pullback/CommSq.lean |
6 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
7-77961 7 days ago |
15-71449 15 days ago |
0-17 17 seconds |
| 30185 |
alreadydone author:alreadydone |
feat(MathlibTest): kernel reduction of nsmul on elliptic curve over ZMod |
Co-authored-by: @SteffenReith
---
- [ ] depends on: #30144
- [x] depends on: #30181
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-algebraic-geometry
t-number-theory
blocked-by-other-PR
label:t-algebra$ |
103/61 |
Mathlib/Algebra/Group/Defs.lean,Mathlib/Algebra/Group/Prod.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Affine/Point.lean,Mathlib/Data/Nat/BinaryRec.lean,Mathlib/Data/Nat/BitIndices.lean,Mathlib/Data/Nat/Bits.lean,Mathlib/Data/Nat/Bitwise.lean,Mathlib/Data/Nat/Digits/Defs.lean,Mathlib/Data/Nat/Size.lean,MathlibTest/EllipticCurve.lean |
10 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
7-74165 7 days ago |
7-76798 7 days ago |
0-1 1 second |
| 29996 |
vihdzp author:vihdzp |
chore(Order/Concept): `IsIntent` and `IsExtent` |
We define predicates for a set to be an intent/extent, and use them to define alternate constructors for a concept. Using these, we golf the complete lattice instances.
---
- [ ] depends on: #30484
[](https://gitpod.io/from-referrer/)
|
t-order
blocked-by-other-PR
|
561/478 |
Mathlib/Algebra/Lie/Submodule.lean,Mathlib/Algebra/Module/Injective.lean,Mathlib/Algebra/Order/Group/Ideal.lean,Mathlib/Algebra/Order/Kleene.lean,Mathlib/Analysis/Convex/Cone/Dual.lean,Mathlib/Analysis/Normed/Group/Seminorm.lean,Mathlib/Analysis/Seminorm.lean,Mathlib/CategoryTheory/Sites/Precoverage.lean,Mathlib/Combinatorics/Digraph/Basic.lean,Mathlib/Combinatorics/SimpleGraph/Basic.lean,Mathlib/Combinatorics/SimpleGraph/Finsubgraph.lean,Mathlib/Combinatorics/SimpleGraph/Subgraph.lean,Mathlib/Combinatorics/Young/YoungDiagram.lean,Mathlib/FieldTheory/Galois/GaloisClosure.lean,Mathlib/GroupTheory/GroupAction/SubMulAction.lean,Mathlib/MeasureTheory/MeasurableSpace/MeasurablyGenerated.lean,Mathlib/ModelTheory/Definability.lean,Mathlib/NumberTheory/NumberField/FractionalIdeal.lean,Mathlib/Order/BooleanAlgebra/Basic.lean,Mathlib/Order/BooleanSubalgebra.lean,Mathlib/Order/CompleteBooleanAlgebra.lean,Mathlib/Order/CompleteLattice/Basic.lean,Mathlib/Order/CompleteLattice/Lemmas.lean,Mathlib/Order/CompleteSublattice.lean,Mathlib/Order/Concept.lean,Mathlib/Order/Disjoint.lean,Mathlib/Order/Heyting/Basic.lean,Mathlib/Order/Heyting/Regular.lean,Mathlib/Order/Hom/Bounded.lean,Mathlib/Order/Hom/BoundedLattice.lean,Mathlib/Order/Hom/Lattice.lean,Mathlib/Order/Interval/Basic.lean,Mathlib/Order/Lattice.lean,Mathlib/Order/Nucleus.lean,Mathlib/Order/Sublattice.lean,Mathlib/Order/UpperLower/CompleteLattice.lean,Mathlib/RingTheory/DedekindDomain/Different.lean,Mathlib/RingTheory/DedekindDomain/Factorization.lean,Mathlib/RingTheory/DedekindDomain/Ideal/Basic.lean,Mathlib/RingTheory/DividedPowers/SubDPIdeal.lean,Mathlib/RingTheory/Filtration.lean,Mathlib/RingTheory/FractionalIdeal/Basic.lean,Mathlib/RingTheory/FractionalIdeal/Extended.lean,Mathlib/RingTheory/FractionalIdeal/Inverse.lean,Mathlib/RingTheory/FractionalIdeal/Operations.lean,Mathlib/RingTheory/GradedAlgebra/Homogeneous/Ideal.lean,Mathlib/Topology/Algebra/Group/ClosedSubgroup.lean,Mathlib/Topology/Algebra/Group/GroupTopology.lean,Mathlib/Topology/Algebra/Module/ClosedSubmodule.lean,Mathlib/Topology/Algebra/OpenSubgroup.lean,Mathlib/Topology/ContinuousMap/Bounded/Normed.lean,Mathlib/Topology/ContinuousMap/CompactlySupported.lean,Mathlib/Topology/ContinuousMap/Ordered.lean,Mathlib/Topology/DiscreteQuotient.lean,Mathlib/Topology/Sets/Closeds.lean,Mathlib/Topology/Sets/Compacts.lean,Mathlib/Topology/Sets/Opens.lean,Mathlib/Topology/Sets/Order.lean |
58 |
25 |
['Vierkantor', 'github-actions', 'linesthatinterlace', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'plp127', 'vihdzp'] |
YaelDillies assignee:YaelDillies |
7-67670 7 days ago |
7-67691 7 days ago |
16-59311 16 days |
| 30255 |
luigi-massacci author:luigi-massacci |
feat(Analysis/Distribution/ContDiffMapSupportedIn): specialize singleton seminorm family for D_K^n when n finite |
Co-authored by: @ADedecker
---
- [ ] depends on: #30253
- [ ] depends on: #30240
- [ ] depends on: #30239
- [ ] depends on: #30236
- [ ] depends on: #30202
- [ ] depends on: #30201
- [ ] depends on: #30199
- [ ] depends on: #30198
- [ ] depends on: #30197
[](https://gitpod.io/from-referrer/)
|
merge-conflict
blocked-by-other-PR
|
476/3 |
Mathlib/Analysis/Distribution/ContDiffMapSupportedIn.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/Data/Set/Function.lean |
3 |
4 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
7-55360 7 days ago |
48-49751 1 month ago |
0-126 2 minutes |
| 30253 |
luigi-massacci author:luigi-massacci |
feat(Analysis/Distribution/ContDiffMapSupportedIn): Add a wrapper for iteratedFDeriv on the type of bundled smooth compactly supported maps |
Add a wrapper for `iteratedFDeriv` and `fderiv` and on `D_K`, specializing the definitions for `D_K^n` for the case `n = \top` .
Co-authored by: @ADedecker
---
- [ ] depends on: #30240
- [ ] depends on: #30239
- [ ] depends on: #30236
- [ ] depends on: #30202
- [ ] depends on: #30201
- [ ] depends on: #30199
- [ ] depends on: #30198
- [ ] depends on: #30197
[](https://gitpod.io/from-referrer/)
|
merge-conflict
blocked-by-other-PR
|
463/18 |
Mathlib/Analysis/Distribution/ContDiffMapSupportedIn.lean |
1 |
4 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
7-51960 7 days ago |
15-74491 15 days ago |
0-599 9 minutes |
| 30375 |
sinhp author:sinhp |
feat(CategoryTheory): Basics of Locally Cartesian Closed Categories |
See https://github.com/leanprover-community/mathlib4/pull/22321
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.
---
- [ ] depends on: #31033
- [ ] depends on: #30373
- [ ] depends on: #31332
[](https://gitpod.io/from-referrer/)
|
t-category-theory
blocked-by-other-PR
WIP
|
1085/0 |
Mathlib.lean,Mathlib/CategoryTheory/LocallyCartesianClosed/Basic.lean,Mathlib/CategoryTheory/LocallyCartesianClosed/ExponentiableMorphism.lean,Mathlib/CategoryTheory/LocallyCartesianClosed/Over.lean,Mathlib/CategoryTheory/LocallyCartesianClosed/Sections.lean |
5 |
7 |
['Jlh18', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'sinhp'] |
nobody |
7-37786 7 days ago |
8-56531 8 days ago |
0-2073 34 minutes |
| 32000 |
Thmoas-Guan author:Thmoas-Guan |
feat(Algebra): projective dimension equal supremum of localized module |
In this PR, we proved that for finitely generated module over Noetherian ring, projective dimension is equal to the supremum of projective dimension of localized modules over all prime/maximal ideals.
---
- [ ] depends on: #31998
[](https://gitpod.io/from-referrer/)
|
blocked-by-other-PR |
349/0 |
Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Localization.lean,Mathlib/RingTheory/LocalProperties/ProjectiveDimension.lean |
3 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
7-17377 7 days ago |
11-8786 11 days ago |
0-55974 15 hours |
| 32033 |
Thmoas-Guan author:Thmoas-Guan |
feat(Algebra): injective dimension equal supremum of localized module |
In this PR, we proved that for module over Noetherian ring, projective dimension is equal to the supremum of injective dimension of localized modules over all prime/maximal ideals.
---
- [ ] depends on: #31995
- [ ] depends on: #31998
[](https://gitpod.io/from-referrer/) |
blocked-by-other-PR |
560/0 |
Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Localization.lean,Mathlib/RingTheory/LocalProperties/Injective.lean,Mathlib/RingTheory/LocalProperties/InjectiveDimension.lean |
4 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
7-17344 7 days ago |
11-8797 11 days ago |
0-366 6 minutes |
| 31999 |
Thmoas-Guan author:Thmoas-Guan |
feat(RingTheory): global dimension equals the supremum over localizations |
Global dimension of ring is equal to supremum of global dimension over localizations at all prime/maximal ideal.
---
- [ ] depends on: #32000
- [ ] depends on: #31998
- [ ] depends on: #29558
[](https://gitpod.io/from-referrer/)
|
awaiting-author
blocked-by-other-PR
|
647/0 |
Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Baer.lean,Mathlib/Algebra/Category/ModuleCat/Localization.lean,Mathlib/RingTheory/GlobalDimension.lean,Mathlib/RingTheory/LocalProperties/ProjectiveDimension.lean |
5 |
n/a |
['Thmoas-Guan', 'github-actions', 'jcommelin', 'mathlib4-dependent-issues-bot'] |
nobody |
7-13694 7 days ago |
unknown |
unknown |
| 29701 |
Thmoas-Guan author:Thmoas-Guan |
feat(Algebra/RingTheory): polynomial over regular ring |
In this PR, we proved that polynomial over regular ring is regular.
---
- [ ] depends on: #28684
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
blocked-by-other-PR
|
326/0 |
Mathlib.lean,Mathlib/RingTheory/RegularLocalRing/Defs.lean,Mathlib/RingTheory/RegularLocalRing/RegularRing/Basic.lean,Mathlib/RingTheory/RegularLocalRing/RegularRing/Polynomial.lean |
4 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
7-10949 7 days ago |
37-2412 1 month ago |
0-10179 2 hours |
| 31046 |
Thmoas-Guan author:Thmoas-Guan |
feat(Homology) : compatibility of map between `Ext` |
In this PR, we proved the compatibility of map between `Ext` induced by exact functor with
1: `mk_0` 2: `comp` 3: `extClass`
---
- [ ] depends on: #31707
[](https://gitpod.io/from-referrer/) |
t-category-theory
blocked-by-other-PR
|
414/0 |
Mathlib.lean,Mathlib/Algebra/Homology/DerivedCategory/ExactFunctor.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/Map.lean,Mathlib/Algebra/Homology/DerivedCategory/ShortExact.lean,Mathlib/Algebra/Homology/HomotopyCategory.lean,Mathlib/Algebra/Homology/HomotopyCategory/Pretriangulated.lean,Mathlib/Algebra/Homology/HomotopyCategory/ShortExact.lean |
7 |
5 |
['Thmoas-Guan', 'github-actions', 'joelriou', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
eric-wieser assignee:eric-wieser |
7-411 7 days ago |
14-71670 14 days ago |
4-2843 4 days |
| 31697 |
Thmoas-Guan author:Thmoas-Guan |
feat(Homology): bijection between `Ext` |
For `F : C ⥤ D` fully faithful functor between abelian category, if one of the following
1: `C` has enough projectives and `F` preserve projective object
2: `D` has enough injectives and `F` preserve injective object
The induced map `Ext X Y n → Ext F(X) F(Y) n` is bijective.
---
- [ ] depends on: #31046
- [ ] depends on: #31696
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-category-theory
blocked-by-other-PR
label:t-algebra$ |
545/0 |
Mathlib.lean,Mathlib/Algebra/Homology/DerivedCategory/ExactFunctor.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/Bijection.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/Map.lean,Mathlib/Algebra/Homology/DerivedCategory/ShortExact.lean,Mathlib/Algebra/Homology/HomotopyCategory.lean,Mathlib/Algebra/Homology/HomotopyCategory/Pretriangulated.lean,Mathlib/Algebra/Homology/HomotopyCategory/ShortExact.lean |
8 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
7-264 7 days ago |
14-68542 14 days ago |
0-1878 31 minutes |
| 31325 |
joelriou author:joelriou |
feat(AlgebraicTopology): a computable monoidal functor instance for `hoFunctor` |
---
- [ ] depends on: #31174
- [x] depends on: #31250
- [x] depends on: #31254
- [x] depends on: #31274
- [x] depends on: #31265
[](https://gitpod.io/from-referrer/)
|
t-algebraic-topology
merge-conflict
blocked-by-other-PR
|
1694/752 |
Mathlib.lean,Mathlib/AlgebraicTopology/SimplicialNerve.lean,Mathlib/AlgebraicTopology/SimplicialSet/Basic.lean,Mathlib/AlgebraicTopology/SimplicialSet/CompStruct.lean,Mathlib/AlgebraicTopology/SimplicialSet/CompStructTruncated.lean,Mathlib/AlgebraicTopology/SimplicialSet/Coskeletal.lean,Mathlib/AlgebraicTopology/SimplicialSet/HoFunctorMonoidal.lean,Mathlib/AlgebraicTopology/SimplicialSet/HomotopyCat.lean,Mathlib/AlgebraicTopology/SimplicialSet/Monoidal.lean,Mathlib/AlgebraicTopology/SimplicialSet/Nerve.lean,Mathlib/AlgebraicTopology/SimplicialSet/NerveAdjunction.lean,Mathlib/AlgebraicTopology/SimplicialSet/Path.lean,Mathlib/AlgebraicTopology/SimplicialSet/StrictSegal.lean,Mathlib/CategoryTheory/Category/ReflQuiv.lean,Mathlib/CategoryTheory/Closed/Cartesian.lean,Mathlib/CategoryTheory/ComposableArrows/Basic.lean,Mathlib/CategoryTheory/Functor/Currying.lean,Mathlib/CategoryTheory/Functor/CurryingThree.lean,Mathlib/CategoryTheory/Monoidal/Cartesian/FunctorCategory.lean,Mathlib/CategoryTheory/MorphismProperty/Basic.lean,Mathlib/CategoryTheory/MorphismProperty/Composition.lean,Mathlib/CategoryTheory/PathCategory/Basic.lean,Mathlib/Combinatorics/Quiver/ReflQuiver.lean |
23 |
5 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
6-86383 6 days ago |
10-46809 10 days ago |
0-2350 39 minutes |
| 31222 |
Thmoas-Guan author:Thmoas-Guan |
feat(Algebra): `Hom` commute with flat base change |
In this PR, we proved `Hom_S (M \tensor S, N \tensor S)` is base change of `Hom_R (M, N)` with respect to `LinearMap.baseChangeHom`.
Co-authored-by: Wang Jingting
---
- [x] depends on: #31218
- [ ] depends on: #31219
- [x] depends on: #31696
[](https://gitpod.io/from-referrer/)
|
large-import
blocked-by-other-PR
|
154/0 |
Mathlib.lean,Mathlib/Algebra/Module/FinitePresentation.lean,Mathlib/RingTheory/Flat/IsBaseChange.lean |
3 |
5 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
6-83824 6 days ago |
6-83832 6 days ago |
0-266 4 minutes |
| 30373 |
sinhp author:sinhp |
feat(CategoryTheory) : LCCC sections (constructing right adjoint to `Over.ChosenPullback.pullback`) |
In LCCCs development, the `sections` functor is used to define the right adjoint to the pullback functor `Over.ChosenPullback.pullback`.
This PR defines `Over.sections` and proves that it is a right adjoint to the `toOver (I : C) : C ⥤ Over I` (this is the computable analogue of `star`).
This is the computable enhancement of #22319: instead of `Limits.pullback` this PR builds on top of `Over.ChosenPullback` and thus we eliminate any instance of noncomputable constructs.
---
- [ ] depends on: #31033
- [ ] depends on: #31433
[](https://gitpod.io/from-referrer/)
|
t-category-theory
blocked-by-other-PR
|
524/0 |
Mathlib.lean,Mathlib/CategoryTheory/Comma/Over/Basic.lean,Mathlib/CategoryTheory/LocallyCartesianClosed/Over.lean,Mathlib/CategoryTheory/LocallyCartesianClosed/Sections.lean |
4 |
9 |
['github-actions', 'joelriou', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'robin-carlier', 'sinhp'] |
robin-carlier assignee:robin-carlier |
6-83684 6 days ago |
8-72264 8 days ago |
0-26856 7 hours |
| 30576 |
smmercuri author:smmercuri |
feat: `adicCompletion` for `Rat` is uniform isomorphic to `Padic` |
---
- [ ] depends on: #30133
- [x] depends on: #30574
- [x] depends on: #30363
- [x] depends on: #30171
- [ ] depends on: #31845
[](https://gitpod.io/from-referrer/)
|
blocked-by-other-PR
WIP
|
246/5 |
Mathlib.lean,Mathlib/Algebra/Order/Hom/Ring.lean,Mathlib/NumberTheory/Padics/HeightOneSpectrum.lean,Mathlib/Topology/Algebra/UniformRing.lean,Mathlib/Topology/Algebra/Valued/WithVal.lean |
5 |
4 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
6-82585 6 days ago |
15-75678 15 days ago |
0-11 11 seconds |
| 32021 |
jsm28 author:jsm28 |
feat(Geometry/Euclidean/Altitude): `map` and `restrict` lemmas |
Add lemmas about `altitude`, `altitudeFoot` and `height` for simplices mapped under an affine isometry or restricted to an affine subspace.
---
- [x] depends on: #32016
- [x] depends on: #32017
- [ ] depends on: #32019
[](https://gitpod.io/from-referrer/)
|
t-euclidean-geometry
blocked-by-other-PR
|
130/0 |
Mathlib/Geometry/Euclidean/Altitude.lean,Mathlib/Geometry/Euclidean/Projection.lean |
2 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
6-71069 6 days ago |
6-71086 6 days ago |
0-87 1 minute |
| 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
merge-conflict
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 |
4 |
['github-actions', 'joelriou', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
6-58122 6 days ago |
63-45262 2 months ago |
0-1160 19 minutes |
| 31919 |
alreadydone author:alreadydone |
feat(RingTheory): integrally closed subring of a field is intersection of valuation subrings |
Co-authored-by: Daniel Funck @danielfunckmaths-commits
This contribution was created as part of the Heidelberg Lean workshop "Formalising algebraic geometry" in November 2025.
---
- [ ] depends on: #32118
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
blocked-by-other-PR
|
273/86 |
Mathlib/Algebra/Algebra/Basic.lean,Mathlib/Algebra/Polynomial/Degree/TrailingDegree.lean,Mathlib/NumberTheory/Padics/PadicIntegers.lean,Mathlib/RingTheory/Ideal/Defs.lean,Mathlib/RingTheory/Ideal/Nonunits.lean,Mathlib/RingTheory/IntegralClosure/IntegrallyClosed.lean,Mathlib/RingTheory/LocalRing/LocalSubring.lean,Mathlib/RingTheory/LocalRing/RingHom/Basic.lean,Mathlib/RingTheory/Polynomial/Basic.lean,Mathlib/RingTheory/Polynomial/Ideal.lean,Mathlib/RingTheory/Valuation/AlgebraInstances.lean,Mathlib/RingTheory/Valuation/Integers.lean,Mathlib/RingTheory/Valuation/LocalSubring.lean,Mathlib/RingTheory/Valuation/ValuationSubring.lean |
14 |
4 |
['alreadydone', 'github-actions', 'jcommelin', 'mathlib4-dependent-issues-bot'] |
nobody |
6-56878 6 days ago |
6-57829 6 days ago |
4-17055 4 days |
| 31135 |
kckennylau author:kckennylau |
feat(RingTheory): is localization iff is localization on saturation |
In this PR we show that `A` is a localization of `R` on the submonoid `S` iff it is so on the saturation of `S`.
Crucially, the saturation of `S` is precisely the elements that become a unit in `A`.
---
- [ ] depends on: #31132
[](https://gitpod.io/from-referrer/)
|
merge-conflict
blocked-by-other-PR
|
293/0 |
Mathlib.lean,Mathlib/Algebra/Group/Submonoid/Saturation.lean,Mathlib/RingTheory/Localization/Saturation.lean |
3 |
5 |
['alreadydone', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
6-54637 6 days ago |
15-86121 15 days ago |
0-169 2 minutes |
| 31954 |
wwylele author:wwylele |
feat(Counterexamples): Weierstrass function is continuous and nowhere differentiable |
---
- [ ] depends on: #31970
- [ ] depends on: #31971
- [ ] depends on: #31973
- [ ] depends on: #31977
- [ ] depends on: #31982
- [ ] depends on: #32082
- [ ] depends on: #32079
[](https://gitpod.io/from-referrer/)
|
blocked-by-other-PR |
345/0 |
Counterexamples.lean,Counterexamples/Weierstrass.lean,docs/references.bib |
3 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
6-50636 6 days ago |
10-18350 10 days ago |
0-0 0 seconds |
| 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
---
- [x] depends on: #27977
- [ ] depends on: #27978
- [x] depends on: #27974
- [x] depends on: #27975
- [ ] depends on: #27976
- [ ] depends on: #29942
- [ ] depends on: #29946 |
large-import
FLT
t-number-theory
merge-conflict
blocked-by-other-PR
|
619/2 |
Mathlib.lean,Mathlib/Analysis/Normed/Field/WithAbs.lean,Mathlib/Analysis/Normed/Ring/WithAbs.lean,Mathlib/NumberTheory/NumberField/Completion.lean,Mathlib/NumberTheory/NumberField/InfinitePlace/Dimension.lean,Mathlib/NumberTheory/NumberField/InfinitePlace/Embeddings.lean,Mathlib/NumberTheory/NumberField/InfinitePlace/Ramification.lean |
7 |
4 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
6-45586 6 days ago |
71-57207 2 months ago |
0-3752 1 hour |
| 31350 |
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 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: #28793 is the first step for this
- [ ] depends on: #31351 defines manifolds with smooth boundary: the main dependence are smooth embeddings (and some basic results about these), then the definition needs redoing.
- depends on: #22874 for some constructions
- defining unoriented bordisms, and proving some basic constructions about them: will be another PR
This PR continues the work from #23138.
|
t-differential-geometry
merge-conflict
blocked-by-other-PR
WIP
|
1084/2 |
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/MFDeriv/SpecificFunctions.lean |
6 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
6-41953 6 days ago |
15-85958 15 days ago |
0-77 1 minute |
| 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 |
6-41870 6 days ago |
87-39110 2 months ago |
0-617 10 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 |
6-41868 6 days ago |
87-39111 2 months ago |
0-11 11 seconds |
| 30240 |
luigi-massacci author:luigi-massacci |
feat(Analysis/Distribution/ContDiffMapSupportedIn): Add a wrapper for fderiv on D_K^n |
Add a wrapper for `fderiv` as a map from `D_K^n` to `D_K^(n-1)`.
Co-Authored by: @ADedecker
---
- [ ] depends on: #30239
- [ ] depends on: #30236
- [ ] depends on: #30202
- [ ] depends on: #30201
- [ ] depends on: #30199
- [ ] depends on: #30198
- [ ] depends on: #30197
[](https://gitpod.io/from-referrer/)
|
t-analysis
blocked-by-other-PR
|
379/16 |
Mathlib/Analysis/Distribution/ContDiffMapSupportedIn.lean |
1 |
6 |
['ADedecker', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
6-38302 6 days ago |
15-75120 15 days ago |
0-546 9 minutes |
| 29274 |
Jlh18 author:Jlh18 |
feat(CategoryTheory): HasLimits instance on Grpd |
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]
- [ ] depends on: #29283
---
[](https://gitpod.io/from-referrer/)
|
file-removed
t-category-theory
blocked-by-other-PR
|
243/65 |
Mathlib.lean,Mathlib/AlgebraicTopology/FundamentalGroupoid/Basic.lean,Mathlib/CategoryTheory/Core.lean,Mathlib/CategoryTheory/Groupoid/FreeGroupoidOfCategory.lean,Mathlib/CategoryTheory/Groupoid/Grpd.lean,Mathlib/CategoryTheory/Groupoid/Grpd/Core.lean,Mathlib/CategoryTheory/Groupoid/Grpd/Free.lean,Mathlib/CategoryTheory/Groupoid/Grpd/Limit.lean,Mathlib/CategoryTheory/Quotient.lean |
9 |
5 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
6-37561 6 days ago |
6-37581 6 days ago |
0-12918 3 hours |
| 32125 |
SnirBroshi author:SnirBroshi |
feat(SimpleGraph/Walks/Subwalks): `p₁.IsSubwalk p₂ ↔ p₁.darts <:+: p₂.darts` and similar theorems |
---
- [ ] depends on: #32160
[](https://gitpod.io/from-referrer/)
|
t-combinatorics
blocked-by-other-PR
|
84/0 |
Mathlib/Combinatorics/SimpleGraph/Walks/Basic.lean,Mathlib/Combinatorics/SimpleGraph/Walks/Subwalks.lean,Mathlib/Combinatorics/SimpleGraph/Walks/Traversal.lean |
3 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
6-27642 6 days ago |
6-27668 6 days ago |
0-83394 23 hours |
| 31560 |
AntoineChambert-Loir author:AntoineChambert-Loir |
feat(Topology/Sion): the minimax theorem of von Neumann - Sion |
Prove `Sion.exists_isSaddlePointOn` :
Let X and Y be convex subsets of topological vector spaces E and F,
X being moreover compact,
and let f : X × Y → ℝ be a function such that
- for all x, f(x, ⬝) is upper semicontinuous and quasiconcave
- for all y, f(⬝, y) is lower semicontinuous and quasiconvex
Then inf_x sup_y f(x,y) = sup_y inf_x f(x,y).
The classical case of the theorem assumes that f is continuous,
f(x, ⬝) is concave, f(⬝, y) is convex.
As a particular case, one get the von Neumann theorem where
f is bilinear and E, F are finite dimensional.
We follow the proof of Komiya (1988).
## Remark on implementation
* The essential part of the proof holds for a function
`f : X → Y → β`, where `β` is a complete dense linear order.
* We have written part of it for just a dense linear order,
* On the other hand, if the theorem holds for such `β`,
it must hold for any linear order, for the reason that
any linear order embeds into a complete dense linear order.
However, this result does not seem to be known to Mathlib.
* When `β` is `ℝ`, one can use `Real.toEReal` and one gets a proof for `ℝ`.
## TODO
Give particular important cases (eg, bilinear maps in finite dimension).
Co-authored with @ADedecker
---
- [ ] depends on: #31548
- [ ] depends on: #31547
- [ ] depends on: #31558
[](https://gitpod.io/from-referrer/)
|
blocked-by-other-PR |
847/1 |
Mathlib.lean,Mathlib/Data/EReal/Basic.lean,Mathlib/Topology/Compactness/Compact.lean,Mathlib/Topology/Semicontinuous.lean,Mathlib/Topology/Sion.lean,Mathlib/Topology/Sublevel.lean,docs/references.bib |
7 |
4 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
5-60215 5 days ago |
5-61634 5 days ago |
0-536 8 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).
---
- [x] depends on: #27567
- [x] depends on: #27569
- [ ] depends on: #32245
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
awaiting-author
blocked-by-other-PR
|
163/0 |
Mathlib.lean,Mathlib/RingTheory/Coalgebra/Frobenius.lean |
2 |
18 |
['YaelDillies', 'erdOne', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'themathqueen'] |
alreadydone assignee:alreadydone |
5-46269 5 days ago |
5-47176 5 days ago |
30-32821 30 days |
| 32260 |
jsm28 author:jsm28 |
feat(Geometry/Euclidean/Angle/Oriented/Affine): oriented angle bisection and halving unoriented angles |
Add lemmas relating points bisecting an oriented angle to explicit expressions for one unoriented angle in relation to half another unoriented angle.
---
Feel free to golf.
---
- [ ] depends on: #32259
[](https://gitpod.io/from-referrer/)
|
t-euclidean-geometry
blocked-by-other-PR
|
277/0 |
Mathlib/Analysis/SpecialFunctions/Trigonometric/Angle.lean,Mathlib/Geometry/Euclidean/Angle/Oriented/Affine.lean |
2 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
5-25225 5 days ago |
5-25226 5 days ago |
0-2532 42 minutes |
| 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
- [x] depends on: #28793
- [x] depends on: #30356
- [ ] depends on: #28853 (for simplicity)
[](https://gitpod.io/from-referrer/)
|
t-differential-geometry
merge-conflict
blocked-by-other-PR
WIP
|
428/33 |
Mathlib/Analysis/Calculus/ContDiff/Basic.lean,Mathlib/Geometry/Manifold/ContMDiff/Atlas.lean,Mathlib/Geometry/Manifold/Immersion.lean,Mathlib/Geometry/Manifold/IsManifold/Basic.lean,Mathlib/Geometry/Manifold/IsManifold/ExtChartAt.lean,Mathlib/Geometry/Manifold/LocalSourceTargetProperty.lean,Mathlib/Topology/OpenPartialHomeomorph.lean,docs/overview.yaml |
8 |
5 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
4-81560 4 days ago |
4-81866 4 days ago |
0-1 1 second |
| 32202 |
joelriou author:joelriou |
feat(AlgebraicTopology): finite simplicial sets |
A simplicial set `X` is finite (`Simplicial.Finite`) if it has finitely many nondegenerate simplices. Equivalently, `X` is finite dimensional and the type of `n`-simplices of `X` is finite for any `n`.
---
- [ ] depends on: #32201
[](https://gitpod.io/from-referrer/)
|
t-algebraic-topology
blocked-by-other-PR
WIP
|
296/0 |
Mathlib.lean,Mathlib/AlgebraicTopology/SimplexCategory/Basic.lean,Mathlib/AlgebraicTopology/SimplicialSet/Dimension.lean,Mathlib/AlgebraicTopology/SimplicialSet/Finite.lean,Mathlib/AlgebraicTopology/SimplicialSet/StdSimplex.lean |
5 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
4-77773 4 days ago |
4-77773 4 days ago |
0-2980 49 minutes |
| 32237 |
joelriou author:joelriou |
feat(AlgebraicTopology): binary products of standard simplices |
We start the study of nondegenerate simplices in `Δ[p] ⊗ Δ[q]`. In particular, we show that it is of dimension `≤ p + q`.
From https://github.com/joelriou/topcat-model-category
---
- [ ] depends on: #32201
- [ ] depends on: #32202
[](https://gitpod.io/from-referrer/)
|
t-algebraic-topology
blocked-by-other-PR
WIP
|
445/0 |
Mathlib.lean,Mathlib/AlgebraicTopology/SimplexCategory/Basic.lean,Mathlib/AlgebraicTopology/SimplicialSet/Dimension.lean,Mathlib/AlgebraicTopology/SimplicialSet/Finite.lean,Mathlib/AlgebraicTopology/SimplicialSet/Monoidal.lean,Mathlib/AlgebraicTopology/SimplicialSet/ProdStdSimplex.lean,Mathlib/AlgebraicTopology/SimplicialSet/StdSimplex.lean |
7 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
4-77766 4 days ago |
4-77766 4 days ago |
0-655 10 minutes |
| 32251 |
joelriou author:joelriou |
feat(AlgebraicTopology): binary products of finite simplicial sets are finite |
If `X₁` and `X₂` are respectively of dimensions `≤ d₁` and `≤ d₂`, then `X₁ ⊗ X₂` has dimension `≤ d₁ + d₂`. We also show that if `X₁` and `X₂` are finite, then `X₁ ⊗ X₂` is also finite.
From https://github.com/joelriou/topcat-model-category
- [ ] depends on: #32201
- [ ] depends on: #32202
- [ ] depends on: #32237
---
[](https://gitpod.io/from-referrer/)
|
t-algebraic-topology
blocked-by-other-PR
WIP
|
578/2 |
Mathlib.lean,Mathlib/AlgebraicTopology/SimplexCategory/Basic.lean,Mathlib/AlgebraicTopology/SimplicialSet/Dimension.lean,Mathlib/AlgebraicTopology/SimplicialSet/Finite.lean,Mathlib/AlgebraicTopology/SimplicialSet/FiniteProd.lean,Mathlib/AlgebraicTopology/SimplicialSet/Monoidal.lean,Mathlib/AlgebraicTopology/SimplicialSet/NonDegenerateSimplices.lean,Mathlib/AlgebraicTopology/SimplicialSet/ProdStdSimplex.lean,Mathlib/AlgebraicTopology/SimplicialSet/StdSimplex.lean |
9 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
4-77759 4 days ago |
4-77759 4 days ago |
0-3312 55 minutes |
| 32265 |
joelriou author:joelriou |
feat(AlgebraicTopology): finite colimits of finite simplicial sets are finite |
From https://github.com/joelriou/topcat-model-category
---
- [ ] depends on: #32201
- [ ] depends on: #32202
[](https://gitpod.io/from-referrer/)
|
t-algebraic-topology
blocked-by-other-PR
WIP
|
378/0 |
Mathlib.lean,Mathlib/AlgebraicTopology/SimplexCategory/Basic.lean,Mathlib/AlgebraicTopology/SimplicialSet/Dimension.lean,Mathlib/AlgebraicTopology/SimplicialSet/Finite.lean,Mathlib/AlgebraicTopology/SimplicialSet/FiniteColimits.lean,Mathlib/AlgebraicTopology/SimplicialSet/StdSimplex.lean,Mathlib/CategoryTheory/FinCategory/Basic.lean |
7 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
4-77295 4 days ago |
4-77752 4 days ago |
0-1203 20 minutes |
| 30129 |
vlad902 author:vlad902 |
feat(SimpleGraph): define and prove basic theory of vertex covers |
Define a predicate `IsVertexCover G C` to state that `C` is a vertex cover of `G`. Furthermore, `G.minVertexCover` is the cardinality of the minimum vertex cover of G. Then prove the basic theory of how these definitions relate to the empty and complete graphs and their relationship with graph homs/isos.
---
- [x] depends on: #29833
- [x] depends on: #30136
- [x] depends on: #30137
- [ ] depends on: #32267
[](https://gitpod.io/from-referrer/)
|
t-combinatorics
blocked-by-other-PR
|
231/3 |
Mathlib.lean,Mathlib/Combinatorics/SimpleGraph/Basic.lean,Mathlib/Combinatorics/SimpleGraph/Clique.lean,Mathlib/Combinatorics/SimpleGraph/Maps.lean,Mathlib/Combinatorics/SimpleGraph/VertexCover.lean |
5 |
57 |
['SnirBroshi', 'YaelDillies', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'vlad902'] |
YaelDillies assignee:YaelDillies |
4-76761 4 days ago |
4-77200 4 days ago |
10-72677 10 days |
| 32270 |
jsm28 author:jsm28 |
feat(Geometry/Euclidean/Incenter): `map` and `restrict` lemmas |
Add lemmas about incenter-related definitions for simplices mapped under an affine isometry or restricted to an affine subspace.
---
- [ ] depends on: #32019
- [ ] depends on: #32021
[](https://gitpod.io/from-referrer/)
|
t-euclidean-geometry
blocked-by-other-PR
|
255/0 |
Mathlib/Geometry/Euclidean/Altitude.lean,Mathlib/Geometry/Euclidean/Incenter.lean,Mathlib/Geometry/Euclidean/Projection.lean |
3 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
4-65532 4 days ago |
4-65533 4 days ago |
0-2817 46 minutes |
| 32273 |
jsm28 author:jsm28 |
feat(Analysis/Convex/Side): affine combinations on same / opposite side of face of a simplex as a vertex |
Build on #31205 by providing lemmas about when an affine combination of the vertices of a simplex is on the same / opposite side of a face (opposite a vertex) of the simplex as that vertex (a specific case of the lemmas from #31205 which involve two arbitrary affine combinations).
---
- [ ] depends on: #31205
[](https://gitpod.io/from-referrer/)
|
t-convex-geometry
t-analysis
blocked-by-other-PR
|
223/0 |
Mathlib/Analysis/Convex/Side.lean |
1 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
4-64414 4 days ago |
4-64415 4 days ago |
0-874 14 minutes |
| 32278 |
jsm28 author:jsm28 |
feat(Geometry/Euclidean/Incenter): excenters on sides of faces |
Add lemmas about when an excenter of a simplex is on the same / opposite side of a face of that simplex (opposite a vertex) as that vertex.
---
- [ ] depends on: #31205
- [ ] depends on: #32273
[](https://gitpod.io/from-referrer/)
|
t-euclidean-geometry
blocked-by-other-PR
|
330/0 |
Mathlib/Analysis/Convex/Side.lean,Mathlib/Geometry/Euclidean/Incenter.lean |
2 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
4-57147 4 days ago |
4-57148 4 days ago |
0-3377 56 minutes |
| 32266 |
joelriou author:joelriou |
feat(AlgebraicTopology): finite simplicial sets are `ℵ₀`-presentable, |
In this file, we show that finite simplicial sets are `ℵ₀`-presentable, which will allow the use of the small object argument in `SSet`.
This PR relaxes the import ban of `SetTheory` in `AlgebraicTopology`: almost all constructions of model category structures require the small object argument.
From https://github.com/joelriou/topcat-model-category
---
- [ ] depends on: #32201
- [ ] depends on: #32202
- [ ] depends on: #32237
- [ ] depends on: #32251
- [ ] depends on: #32265
- [ ] depends on: #32279
[](https://gitpod.io/from-referrer/)
|
t-algebraic-geometry
blocked-by-other-PR
WIP
|
965/3 |
Mathlib.lean,Mathlib/AlgebraicTopology/SimplexCategory/Basic.lean,Mathlib/AlgebraicTopology/SimplicialSet/Dimension.lean,Mathlib/AlgebraicTopology/SimplicialSet/Finite.lean,Mathlib/AlgebraicTopology/SimplicialSet/FiniteColimits.lean,Mathlib/AlgebraicTopology/SimplicialSet/FiniteProd.lean,Mathlib/AlgebraicTopology/SimplicialSet/Monoidal.lean,Mathlib/AlgebraicTopology/SimplicialSet/NonDegenerateSimplices.lean,Mathlib/AlgebraicTopology/SimplicialSet/Presentable.lean,Mathlib/AlgebraicTopology/SimplicialSet/ProdStdSimplex.lean,Mathlib/AlgebraicTopology/SimplicialSet/StdSimplex.lean,Mathlib/CategoryTheory/Comma/CardinalArrow.lean,Mathlib/CategoryTheory/EffectiveEpi/Coequalizer.lean,Mathlib/CategoryTheory/EffectiveEpi/FunctorToTypes.lean,Mathlib/CategoryTheory/FinCategory/Basic.lean,Mathlib/CategoryTheory/Limits/Shapes/Pullback/CommSq.lean,Mathlib/CategoryTheory/Limits/Types/Coequalizers.lean,Mathlib/CategoryTheory/Limits/Types/EffectiveEpi.lean,Mathlib/CategoryTheory/Limits/Types/Pullbacks.lean,Mathlib/Tactic/Linter/DirectoryDependency.lean |
20 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
4-53221 4 days ago |
4-57212 4 days ago |
0-1 1 second |
| 32282 |
jsm28 author:jsm28 |
feat(Geometry/Euclidean/Angle/Incenter): unoriented angle bisection |
Add lemmas giving unoriented angles involving the incenter and excenters of a triangle as expressions involving dividing angles of the triangle by 2, deduced from oriented bisection lemmas.
---
- [ ] depends on: #30981
- [ ] depends on: #30982
- [ ] depends on: #31205
- [ ] depends on: #32019
- [ ] depends on: #32021
- [ ] depends on: #32259
- [ ] depends on: #32260
- [ ] depends on: #32270
- [ ] depends on: #32273
- [ ] depends on: #32278
[](https://gitpod.io/from-referrer/)
|
t-euclidean-geometry
blocked-by-other-PR
|
1380/4 |
Mathlib.lean,Mathlib/Analysis/Convex/Side.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Angle.lean,Mathlib/Geometry/Euclidean/Altitude.lean,Mathlib/Geometry/Euclidean/Angle/Bisector.lean,Mathlib/Geometry/Euclidean/Angle/Incenter.lean,Mathlib/Geometry/Euclidean/Angle/Oriented/Affine.lean,Mathlib/Geometry/Euclidean/Incenter.lean,Mathlib/Geometry/Euclidean/Projection.lean |
9 |
n/a |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
4-52887 4 days ago |
unknown |
unknown |
| 31495 |
jsm28 author:jsm28 |
feat(Geometry/Euclidean/Sphere/SecondInter): `secondInter` and sides of faces of a simplex |
Add lemmas that, if you take a simplex with one vertex on a sphere and the others on or inside it (typically, a triangle and its circumcircle), and take a line through the given vertex and a point in the interior of the simplex or the interior of the opposite face, the second intersection of that line with the sphere lies on the opposite side (from the vertex) of the face opposite that vertex.
---
- [ ] depends on: #31451
- [ ] depends on: #31452
[](https://gitpod.io/from-referrer/)
|
t-euclidean-geometry
blocked-by-other-PR
|
217/0 |
Mathlib.lean,Mathlib/Analysis/Convex/StrictCombination.lean,Mathlib/Geometry/Euclidean/Sphere/SecondInter.lean |
3 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
4-31963 4 days ago |
15-76466 15 days ago |
0-336 5 minutes |
| 30327 |
luigi-massacci author:luigi-massacci |
feat(Analysis/Distribution/TestFunction): add characterizations of continuity for linear maps on test functions |
---
- [ ] depends on: #31806
- [x] depends on: #30309
- [x] depends on: #31470
- [ ] depends on: #30255
- [ ] depends on: #30253
- [ ] depends on: #30240
- [ ] depends on: #30239
- [x] depends on: #30236
- [x] depends on: #30202
- [x] depends on: #30201
- [x] depends on: #30199
- [x] depends on: #30198
- [x] depends on: #30197
[](https://gitpod.io/from-referrer/)
|
merge-conflict
blocked-by-other-PR
|
774/5 |
Mathlib.lean,Mathlib/Analysis/Distribution/ContDiffMapSupportedIn.lean,Mathlib/Analysis/Distribution/TestFunction.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/Data/Set/Function.lean |
5 |
4 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
3-80503 3 days ago |
48-49746 1 month ago |
0-64 1 minute |
| 31892 |
jsm28 author:jsm28 |
feat(Geometry/Euclidean/Sphere/PolePolar): poles and polars |
Define poles and polars for spheres in Euclidean affine spaces, and set up some basic API, including in particular La Hire's theorem (`p₁` lies on the polar of `p₂` if and only if `p₂` lies on the polar of `p₁`).
Poles and polars are actually meaningful for any quadric in a projective space over any field, but I think it's reasonable to set up this theory for spheres in the Euclidean context and potentially link it in future to more general projective geometry.
---
- [ ] depends on: #31891
- [ ] depends on: #32296
[](https://gitpod.io/from-referrer/)
|
t-euclidean-geometry
blocked-by-other-PR
|
246/1 |
Mathlib.lean,Mathlib/Geometry/Euclidean/Sphere/OrthRadius.lean,Mathlib/Geometry/Euclidean/Sphere/PolePolar.lean |
3 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
3-71004 3 days ago |
13-70233 13 days ago |
0-760 12 minutes |
| 31893 |
jsm28 author:jsm28 |
feat(Geometry/Euclidean/Sphere/Tangent): characterize `tangentsFrom` |
Add lemmas relating tangency to polars, and thereby characterizing `tangentsFrom`: empty for a point inside the sphere, a singleton for a point on the sphere and, in two dimensions, of cardinality two for a point outside the circle.
---
- [ ] depends on: #31891
- [ ] depends on: #31892
- [ ] depends on: #32296
[](https://gitpod.io/from-referrer/)
|
t-euclidean-geometry
blocked-by-other-PR
|
305/3 |
Mathlib.lean,Mathlib/Geometry/Euclidean/Sphere/OrthRadius.lean,Mathlib/Geometry/Euclidean/Sphere/PolePolar.lean,Mathlib/Geometry/Euclidean/Sphere/Tangent.lean |
4 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
3-70953 3 days ago |
13-70235 13 days ago |
0-313 5 minutes |
| 31981 |
jsm28 author:jsm28 |
feat(Geometry/Euclidean/Incenter): `tangentSet` and `tangentsFrom` lemmas |
Add lemmas relating the faces of a simplex to `tangentSet` and `tangentsFrom` for an exsphere, in particular for a triangle that any two side lines are the `tangentsFrom` their shared vertex to the insphere or any exsphere.
---
- [ ] depends on: #31733
- [ ] depends on: #31891
- [ ] depends on: #31892
- [ ] depends on: #31893
- [x] depends on: #31978
- [ ] depends on: #31979
- [x] depends on: #31980
- [ ] depends on: #32296
[](https://gitpod.io/from-referrer/)
|
t-euclidean-geometry
blocked-by-other-PR
|
510/3 |
Mathlib.lean,Mathlib/Geometry/Euclidean/Incenter.lean,Mathlib/Geometry/Euclidean/Sphere/OrthRadius.lean,Mathlib/Geometry/Euclidean/Sphere/PolePolar.lean,Mathlib/Geometry/Euclidean/Sphere/Tangent.lean,Mathlib/LinearAlgebra/AffineSpace/Independent.lean |
6 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
3-70941 3 days ago |
12-22545 12 days ago |
0-1725 28 minutes |
| 32307 |
mcdoll author:mcdoll |
feat(Analysis/Distribution): `(1 + |x|^2)^r` has temperate growth |
---
- [ ] depends on: #32297
[](https://gitpod.io/from-referrer/)
|
t-analysis
blocked-by-other-PR
WIP
|
166/2 |
Mathlib/Analysis/Distribution/SchwartzSpace.lean,Mathlib/Analysis/Distribution/TemperateGrowth.lean |
2 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
3-64346 3 days ago |
3-64347 3 days ago |
0-31 31 seconds |
| 32308 |
joelriou author:joelriou |
feat(Algebra/Homology): the bifunctor `F.map₂CochainComplex` commutes with shifts |
Let `F : C₁ ⥤ C₂ ⥤ D` be a bifunctor (which is additive in both variables). In this PR, we show that the induced bifunctor `F.map₂CochainComplex : CochainComplex C₁ ℤ ⥤ CochainComplex C₂ ℤ ⥤ CochainComplex D ℤ` commutes with shifts by `ℤ`. (This means that it commutes with shifts by each variable, and also that there is a commutativity up to a sign when we consider both commutation at the same time.)
---
- [ ] depends on: #32303
[](https://gitpod.io/from-referrer/)
|
t-category-theory
blocked-by-other-PR
WIP
|
333/4 |
Mathlib.lean,Mathlib/Algebra/Homology/Bifunctor.lean,Mathlib/Algebra/Homology/BifunctorShift.lean,Mathlib/CategoryTheory/Center/NegOnePow.lean,Mathlib/CategoryTheory/Shift/CommShiftTwo.lean,Mathlib/CategoryTheory/Shift/Twist.lean |
6 |
4 |
['github-actions', 'joelriou', 'mathlib4-dependent-issues-bot'] |
nobody |
3-60112 3 days ago |
3-60120 3 days ago |
0-1 1 second |
| 32317 |
joelriou author:joelriou |
feat(CategoryTheory): natural transformations between bifunctors which commute to shifts in two variables |
We introduce the two variable counterpart `NatTrans.CommShift₂` of `NatTrans.CommShift`. We also define `Functor.CommShift₂` instances for the precomposition on each variable.
---
- [ ] depends on: #32303
[](https://gitpod.io/from-referrer/)
|
t-category-theory
blocked-by-other-PR
WIP
|
240/1 |
Mathlib.lean,Mathlib/CategoryTheory/Center/NegOnePow.lean,Mathlib/CategoryTheory/Functor/Category.lean,Mathlib/CategoryTheory/Shift/CommShiftTwo.lean,Mathlib/CategoryTheory/Shift/Twist.lean |
5 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
3-55311 3 days ago |
3-55312 3 days ago |
0-1 1 second |
| 32319 |
urkud author:urkud |
feat: add `ContDiffAt.continuousAt_fderiv` etc |
---
- [ ] depends on: #32318
[](https://gitpod.io/from-referrer/)
|
t-analysis
blocked-by-other-PR
|
77/20 |
Mathlib/Analysis/Calculus/ContDiff/Basic.lean,Mathlib/Topology/Algebra/Module/LinearMap.lean,Mathlib/Topology/Algebra/Module/StrongTopology.lean |
3 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
3-40097 3 days ago |
3-40097 3 days ago |
0-2492 41 minutes |
| 30532 |
Thmoas-Guan author:Thmoas-Guan |
feat(Homology) : `Ext` commute with flat base change |
In this PR, using the linear map `Ext(M,N) => Ext(F(M), F(N))` when `F` is exact functor, we prove that `Ext` commute with flat base change if the ring is noetherian and two modules are finitely generated, stated using `IsBaseChange`
---
- [x] depends on: #27416
- [ ] depends on: #31046
- [ ] depends on: #31222
[](https://gitpod.io/from-referrer/)
|
large-import
t-category-theory
merge-conflict
blocked-by-other-PR
|
1065/0 |
Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Ext/BaseChange.lean,Mathlib/Algebra/Homology/DerivedCategory/ExactFunctor.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/Map.lean,Mathlib/Algebra/Homology/DerivedCategory/ShortExact.lean,Mathlib/Algebra/Homology/HomotopyCategory.lean,Mathlib/Algebra/Homology/HomotopyCategory/Pretriangulated.lean,Mathlib/Algebra/Homology/HomotopyCategory/ShortExact.lean,Mathlib/Algebra/Module/Equiv/Basic.lean,Mathlib/Algebra/Module/FinitePresentation.lean,Mathlib/RingTheory/Flat/IsBaseChange.lean |
11 |
n/a |
['Thmoas-Guan', 'github-actions', 'joelriou', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
3-20021 3 days ago |
unknown |
unknown |
| 32171 |
Thmoas-Guan author:Thmoas-Guan |
feat(RingTheory): polynomial over Gorenstein ring is Gorenstein |
In this PR, we prove that polynomial over Gorenstein ring is Gorenstein.
---
- [ ] depends on: #30532
- [ ] depends on: #31884
- [ ] depends on: #32098
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
large-import
merge-conflict
blocked-by-other-PR
|
2733/0 |
Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Baer.lean,Mathlib/Algebra/Category/ModuleCat/Ext/BaseChange.lean,Mathlib/Algebra/Category/ModuleCat/Ext/Finite.lean,Mathlib/Algebra/Category/ModuleCat/Ext/Ulift.lean,Mathlib/Algebra/Category/ModuleCat/InjectiveDimension.lean,Mathlib/Algebra/Category/ModuleCat/Ulift.lean,Mathlib/Algebra/Homology/DerivedCategory/ExactFunctor.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/Bijection.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/Map.lean,Mathlib/Algebra/Homology/DerivedCategory/ShortExact.lean,Mathlib/Algebra/Homology/HomotopyCategory.lean,Mathlib/Algebra/Homology/HomotopyCategory/Pretriangulated.lean,Mathlib/Algebra/Homology/HomotopyCategory/ShortExact.lean,Mathlib/Algebra/Module/Equiv/Basic.lean,Mathlib/Algebra/Module/FinitePresentation.lean,Mathlib/RingTheory/Flat/IsBaseChange.lean,Mathlib/RingTheory/Gorenstein/Defs.lean,Mathlib/RingTheory/Gorenstein/Polynomial.lean,Mathlib/RingTheory/Regular/InjectiveDimension.lean |
20 |
n/a |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
3-19525 3 days ago |
unknown |
unknown |
| 30204 |
yonggyuchoimath author:yonggyuchoimath |
feat(Algebra/Category/Ring/EqualizerPushout): add effectiveEpi_of_faithfullyFlat in CommRingCatᵒᵖ |
This PR proves that any map `f : S ⟶ R` in `CommRingCatᵒᵖ` with faithfully flat `f.unop : R.unop ⟶ S.unop` is
an effective epimorphism.
Main results:
- `CommRingCat.Equalizer.isLimitForkPushoutSelfOfFaithfullyFlat` : If `f : R ⟶ S` is a faithfully flat map in `CommRingCat`, then `Fork.ofι f pushout.condition` is an equalizer diagram.
- `CommRingCat.Opposite.effectiveEpi_of_faithfullyFlat` : Any map `f : S ⟶ R` in `CommRingCatᵒᵖ` with faithfully flat `f.unop : R.unop ⟶ S.unop` is an effective epimorphism.
---
- [ ] depends on: #29960
- [x] depends on: #30200 |
blocked-by-other-PR |
406/1 |
Mathlib.lean,Mathlib/Algebra/Category/Ring/EqualizerPushout.lean,Mathlib/LinearAlgebra/TensorProduct/Tower.lean,Mathlib/RingTheory/TensorProduct/IncludeLeftSubRight.lean,Mathlib/RingTheory/TensorProduct/Maps.lean |
5 |
5 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
3-7735 3 days ago |
3-13433 3 days ago |
0-1375 22 minutes |
| 28462 |
joelriou author:joelriou |
feat(AlgebraicTopology/SimplicialSet): the relative cell complex attached to a rank function for a pairing |
---
- [ ] depends on: #31122
- [ ] depends on: #28351
- [ ] depends on: #28346
- [ ] depends on: #28336
- [x] depends on: #28332
- [x] depends on: #28330
- [x] depends on: #28224
- [x] depends on: #27968
- [x] depends on: #28034
- [x] depends on: #26076
[](https://gitpod.io/from-referrer/)
|
t-algebraic-topology
blocked-by-other-PR
WIP
|
793/0 |
Mathlib.lean,Mathlib/AlgebraicTopology/SimplexCategory/Basic.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/Subcomplex.lean |
8 |
5 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
3-1671 3 days ago |
30-68603 1 month ago |
0-1 1 second |
| 32347 |
joelriou author:joelriou |
feat(AlgebraicTopology/SimplicialSet): structures to study homotopy groups of Kan complexes |
We introduce a structure `SSet.PtSimplex` which consists of morphisms `Δ[n] ⟶ X` which are constant to a certain `x : X _⦋0⦌` on boundary. Homotopy groups of Kan complexes will be defined as a quotient of this. We introduce two structures `PtSimplex.RelStruct` and `PtSimplex.MulStruct` which will be important in the study of homotopy groups of Kan complexes.
From https://github.com/joelriou/topcat-model-category
---
- [ ] depends on: #32345
[](https://gitpod.io/from-referrer/)
|
t-algebraic-topology
blocked-by-other-PR
|
303/1 |
Mathlib.lean,Mathlib/AlgebraicTopology/SimplicialSet/KanComplex/MulStruct.lean,Mathlib/AlgebraicTopology/SimplicialSet/Monoidal.lean,Mathlib/AlgebraicTopology/SimplicialSet/RelativeMorphism.lean,Mathlib/AlgebraicTopology/SimplicialSet/Subcomplex.lean |
5 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
2-79183 2 days ago |
2-84089 2 days ago |
0-108 1 minute |
| 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
- [x] depends on: #29322
- [ ] depends on: #32045 |
t-ring-theory
blocked-by-other-PR
|
347/125 |
Mathlib/NumberTheory/RamificationInertia/Basic.lean,Mathlib/RingTheory/Localization/AtPrime/Basic.lean,Mathlib/RingTheory/Localization/AtPrime/Extension.lean,Mathlib/RingTheory/Trace/Quotient.lean |
4 |
6 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
2-77030 2 days ago |
2-77030 2 days ago |
0-1979 32 minutes |
| 30927 |
callesonne author:callesonne |
feat(Bicategory/Yoneda): add the yoneda pseudofunctor |
---
- [ ] depends on: #30926
- [x] depends on: #30895
- [x] depends on: #25901
[](https://gitpod.io/from-referrer/)
|
blocked-by-other-PR |
187/17 |
Mathlib.lean,Mathlib/CategoryTheory/Bicategory/Basic.lean,Mathlib/CategoryTheory/Bicategory/FunctorBicategory/Oplax.lean,Mathlib/CategoryTheory/Bicategory/FunctorBicategory/Pseudo.lean,Mathlib/CategoryTheory/Bicategory/NaturalTransformation/Oplax.lean,Mathlib/CategoryTheory/Bicategory/Yoneda.lean,Mathlib/CategoryTheory/Category/Cat.lean,Mathlib/Data/Opposite.lean |
8 |
n/a |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
2-73048 2 days ago |
unknown |
unknown |
| 31364 |
YaelDillies author:YaelDillies |
feat: binomial random graphs |
From LeanCamCombi and formal-conjectures
---
- [x] depends on: #31391
- [x] depends on: #31392
- [x] depends on: #31393
- [x] depends on: #31394
- [x] depends on: #31396
- [x] depends on: #31397
- [x] depends on: #31398
- [x] depends on: #31442
- [x] depends on: #31443
- [x] depends on: #31445
- [ ] depends on: #31908
[](https://gitpod.io/from-referrer/)
|
t-measure-probability
t-combinatorics
blocked-by-other-PR
|
310/7 |
Mathlib.lean,Mathlib/Probability/Combinatorics/BinomialRandomGraph/Defs.lean,Mathlib/Probability/Combinatorics/README.md,Mathlib/Probability/Distributions/Bernoulli.lean,Mathlib/Probability/HasLaw.lean |
5 |
9 |
['LibertasSpZ', 'YaelDillies', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
EtienneC30 assignee:EtienneC30 |
2-57631 2 days ago |
13-53569 13 days ago |
5-83680 5 days |
| 30811 |
yonggyuchoimath author:yonggyuchoimath |
feat(AlgebraicGeometry.EffectiveEpi): effective epimorphisms in schemes |
We prove the following:
* `AffineScheme.effectiveEpiOfFlatOfSurjective`: A flat surjective morphism (between affine schemes) is an effective epimorphism in the category of affine schemes.
* `descSpecOfFlatOfSurjective`: Given a morphism `e : Spec S ⟶ U` of schemes which coequalizes the two projections `(Spec S) ×[Spec R] (Spec S) ⟶ Spec S`, this constructs a unique morphism `Spec R ⟶ U` of schemes that `e` factors through.
* `effectiveEpi_Spec_of_flat_of_surjective`: If `f : R ⟶ S` is a flat ring map in `CommRingCat` with surjective `Spec.map f : Spec S ⟶ Spec R`, then `Spec.map f : Spec S ⟶ Spec R` is an effective epimorphism in the category of schemes.
---
- [x] depends on: #30237
- [ ] depends on: #30204
Note:
I've again incorporated `Scheme.isAffine_local_affine`, an instance saying that any `Scheme.local_affine` at a point gives an affine scheme, in order to define `coverR` in line 259. As already noted in [this review](https://github.com/leanprover-community/mathlib4/pull/30034#pullrequestreview-3277376677) of #30034, having `Scheme.local_affine` in statements is not desirable as any such statements should be true for any open affine neightborhoods.
In fact, it is possible to define `coverR` (and prove the rest) without invoking this instance, e.g., using [`exists_isAffineOpen_mem_and_subset`](https://leanprover-community.github.io/mathlib4_docs/Mathlib/AlgebraicGeometry/AffineScheme.html#AlgebraicGeometry.exists_isAffineOpen_mem_and_subset). A problem of this approach is that `IsAffine` is not automatically synthesized (even if I add an `IsAffine` instance for `exists_isAffineOpen_mem_and_subset`) because `hxU : x ∈ U` can't be synthesized automatically, and this forced to explicitly write down the proof of `IsAffine` everytime. That's the reason that I included `Scheme.isAffine_local_affine` in this PR. I would appreciate any suggestions on this.
Another note:
I've marked many definitions and lemmas with `private`. My criterion was the following:
- It is not optimal as it is stated and can be enhanced after proving `effectiveEpi_Spec_of_flat_of_surjective`: `base_factorization` in line 102 (as it should be true for quasi-compact coverings that are flat surjective).
- The definition/lemma seems specific to the proof of `descSpecOfFlatOfSurjective`. Even when proving fpqc morphisms of algebraic spaces are effective epimorphisms, we would only need `descSpecOfFlatOfSurjective` and lemmas about it (but not the things like `e'_coeq_pullback_f'` or `desc'_cocycle_condition`), cf. [Stacks project, Tag 04P2](https://stacks.math.columbia.edu/tag/04P2). |
blocked-by-other-PR |
792/1 |
Mathlib.lean,Mathlib/Algebra/Category/Ring/EqualizerPushout.lean,Mathlib/AlgebraicGeometry/AffineScheme.lean,Mathlib/AlgebraicGeometry/EffectiveEpi.lean,Mathlib/LinearAlgebra/TensorProduct/Tower.lean,Mathlib/RingTheory/TensorProduct/IncludeLeftSubRight.lean,Mathlib/RingTheory/TensorProduct/Maps.lean |
7 |
4 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
2-55337 2 days ago |
2-56169 2 days ago |
0-2336 38 minutes |
| 31138 |
AntoineChambert-Loir author:AntoineChambert-Loir |
feat(LinearAlgebra/Transvection): the determinant of transvection in a module is equal to 1 |
Proof that the determinant of a transvection is equal to 1.
The proof goes by showing that the determinant of `LinearMap.transvection f v` is `1 + f v` (even if `f v` is nonzero).
I first treat the case of a field, distinguishing whether `f v = 0` (so that we get
a transvection) or not (so that we have a dilation).
Then, by base change to the field of fractions, I can handle the case of a domain. Finally, the general case is treated by base change from the “universal case” where the base ring is the ring of polynomials in $$2n$$ indeterminates corresponding to the coefficients of $$f$$ and $$v$$.
---
- [ ] depends on: #31164
- [ ] depends on: #31165
- [ ] depends on: #30987
- [ ] depends on: #31078
- [ ] depends on: #31162
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebra
blocked-by-other-PR
label:t-algebra$ |
595/26 |
Mathlib/Algebra/Polynomial/RingDivision.lean,Mathlib/LinearAlgebra/Determinant.lean,Mathlib/LinearAlgebra/DirectSum/Finsupp.lean,Mathlib/LinearAlgebra/Finsupp/LinearCombination.lean,Mathlib/LinearAlgebra/SpecialLinearGroup.lean,Mathlib/LinearAlgebra/Transvection.lean,Mathlib/RingTheory/TensorProduct/IsBaseChangeFree.lean,Mathlib/RingTheory/TensorProduct/IsBaseChangeHom.lean |
8 |
9 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'ocfnash'] |
nobody |
2-52874 2 days ago |
2-84481 2 days ago |
0-26 26 seconds |
| 32027 |
alreadydone author:alreadydone |
feat(Counterexamples): invertible module not isomorphic to any ideal |
---
- [ ] depends on: #30736
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
merge-conflict
blocked-by-other-PR
|
495/89 |
Counterexamples.lean,Counterexamples/InvertibleModuleNotIdeal.lean,Mathlib/Algebra/Algebra/Bilinear.lean,Mathlib/Algebra/Algebra/Operations.lean,Mathlib/Algebra/TrivSqZeroExt.lean,Mathlib/Data/Set/Semiring.lean,Mathlib/LinearAlgebra/Span/Defs.lean,Mathlib/RingTheory/ClassGroup.lean,Mathlib/RingTheory/FractionalIdeal/Basic.lean,Mathlib/RingTheory/FractionalIdeal/Operations.lean,Mathlib/RingTheory/Localization/Defs.lean,Mathlib/RingTheory/PicardGroup.lean,docs/references.bib |
13 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
2-39697 2 days ago |
5-79419 5 days ago |
0-2995 49 minutes |
| 30931 |
Thmoas-Guan author:Thmoas-Guan |
feat(RingTheory): Gorenstein local ring is Cohen Macaulay |
In this PR, we give the definition of Gorenstein local ring and proved it is Cohen--Macaulay.
---
- [ ] depends on: #30532
- [ ] depends on: #26218
- [ ] depends on: #29670
[](https://gitpod.io/from-referrer/)
|
large-import
merge-conflict
blocked-by-other-PR
|
5567/28 |
Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Baer.lean,Mathlib/Algebra/Category/ModuleCat/Ext/BaseChange.lean,Mathlib/Algebra/Category/ModuleCat/Ext/Finite.lean,Mathlib/Algebra/Category/ModuleCat/Ext/Ulift.lean,Mathlib/Algebra/Category/ModuleCat/InjectiveDimension.lean,Mathlib/Algebra/Category/ModuleCat/Localization.lean,Mathlib/Algebra/Category/ModuleCat/Ulift.lean,Mathlib/Algebra/Homology/DerivedCategory/ExactFunctor.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/Bijection.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/Map.lean,Mathlib/Algebra/Homology/DerivedCategory/ShortExact.lean,Mathlib/Algebra/Homology/HomotopyCategory.lean,Mathlib/Algebra/Homology/HomotopyCategory/Pretriangulated.lean,Mathlib/Algebra/Homology/HomotopyCategory/ShortExact.lean,Mathlib/Algebra/Module/Equiv/Basic.lean,Mathlib/Algebra/Module/FinitePresentation.lean,Mathlib/CategoryTheory/Abelian/Projective/Dimension.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/RingTheory/CohenMacaulay/Basic.lean,Mathlib/RingTheory/Flat/IsBaseChange.lean,Mathlib/RingTheory/Gorenstein/CohenMacaulay.lean,Mathlib/RingTheory/Gorenstein/Defs.lean,Mathlib/RingTheory/Ideal/AssociatedPrime/Localization.lean,Mathlib/RingTheory/Regular/Category.lean,Mathlib/RingTheory/Regular/Depth.lean,Mathlib/RingTheory/Regular/InjectiveDimension.lean,Mathlib/RingTheory/Regular/Ischebeck.lean,Mathlib/RingTheory/Regular/ProjectiveDimension.lean |
29 |
n/a |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
2-3037 2 days ago |
unknown |
unknown |
| 26291 |
RemyDegenne author:RemyDegenne |
feat(Probability): Cameron-Martin theorem |
- 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
- [x] depends on: #28343
- [x] depends on: #30167
- [x] depends on: #30346
- [ ] depends on: #30348
- [ ] depends on: #30582
[](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
|
1963/13 |
Mathlib.lean,Mathlib/MeasureTheory/Function/ConvergenceInDistribution.lean,Mathlib/MeasureTheory/Measure/Portmanteau.lean,Mathlib/Probability/Distributions/Gaussian/CameronMartin.lean,Mathlib/Probability/Distributions/Gaussian/CameronMartinThm.lean,Mathlib/Probability/Distributions/Gaussian/CompletionResultsToBeMoved.lean,Mathlib/Probability/Distributions/Gaussian/Real.lean,Mathlib/Probability/Moments/CovarianceBilinDual.lean,Mathlib/Probability/Moments/Variance.lean,Mathlib/Topology/Algebra/Module/Basic.lean,Mathlib/Topology/Algebra/Module/ClosedSubmodule.lean,Mathlib/Topology/EMetricSpace/Lipschitz.lean,Mathlib/Topology/UniformSpace/AbstractCompletion.lean,docs/1000.yaml |
14 |
10 |
['github-actions', 'grunweg', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
1-66099 1 day ago |
56-57959 1 month ago* |
0-2 2 seconds* |
| 31749 |
YaelDillies author:YaelDillies |
refactor: make `LinearOrderedCommMonoidWithZero`s cancellative |
It appears that the only interesting `LinearOrderedCommMonoidWithZero`s are the ones for which every non-zero element is regular. This PR therefore strenghtens `LinearOrderedCommMonoidWithZero`, and similarly for `LinearOrderedAddCommMonoidWithTop`, its additive counterpart.
Here are the instances we lose:
* `ENNReal`: multiplication by `\top` isn't injective
* `ERealᵒᵈ`: multiplication by `\top` isn't injective
* `Cardinal`: multiplication by anything but 1 isn't injective
* `ArchimedeanClass R` where `R` is a non-strict ordered ring
* the pathological counterexample of a `LinearOrderedCommMonoidWithZero` where two positive numbers multiply to zero
I believe these are all fine to lose since they had no mathematical motivation (we never use those as targets of valuations).
There is an argument to be made that we could keep the existing typeclass as is and instead have the one I'm currently replacing it with under the name `LinearOrderedCancelCommMonoidWithZero`. There are at least two reasons I do not want to do this:
1. We have no evidence that the weaker typeclass is actually useful
2. `LinearOrderedCommMonoidWithZero`, weak or strong version, extends both the algebra and order hierarchy, which is something we want to move away from. Therefore, if anything, we should not be adding more of those typeclasses.
This will be used in a later PR to replace `pow_eq_one_iff` with `IsMulTorsionFree.pow_eq_one_iff_left`.
[Zulip](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Should.20linear.20ordered.20comm.20monoids.20with.20zero.20be.20torsion-free)
---
- [x] depends on: #31739
- [x] depends on: #31765
- [x] depends on: #31783
- [x] depends on: #31883
- [x] depends on: #31890
- [x] depends on: #31894
- [x] depends on: #31895
- [ ] depends on: #32382
[](https://gitpod.io/from-referrer/)
|
file-removed
large-import
t-algebra
blocked-by-other-PR
label:t-algebra$ |
271/400 |
Counterexamples.lean,Counterexamples/LinearOrderWithPosMulPosEqZero.lean,Mathlib/Algebra/Order/AddGroupWithTop.lean,Mathlib/Algebra/Order/Field/Canonical.lean,Mathlib/Algebra/Order/GroupWithZero/Canonical.lean,Mathlib/Algebra/Order/Nonneg/Ring.lean,Mathlib/Algebra/Order/PUnit.lean,Mathlib/Algebra/Order/Ring/Archimedean.lean,Mathlib/Algebra/Order/Ring/Nat.lean,Mathlib/Data/ENNReal/Basic.lean,Mathlib/Data/ENNReal/Real.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/Data/EReal/Operations.lean,Mathlib/Data/Nat/PartENat.lean,Mathlib/LinearAlgebra/Dimension/Finite.lean,Mathlib/MeasureTheory/Function/ConditionalExpectation/Real.lean,Mathlib/MeasureTheory/Function/ConvergenceInMeasure.lean,Mathlib/MeasureTheory/Integral/Bochner/Basic.lean,Mathlib/MeasureTheory/Integral/Bochner/Set.lean,Mathlib/MeasureTheory/Integral/Lebesgue/Basic.lean,Mathlib/MeasureTheory/Measure/Decomposition/Exhaustion.lean,Mathlib/MeasureTheory/Measure/Doubling.lean,Mathlib/MeasureTheory/Measure/EverywherePos.lean,Mathlib/MeasureTheory/Measure/LevyProkhorovMetric.lean,Mathlib/MeasureTheory/Measure/TightNormed.lean,Mathlib/MeasureTheory/OuterMeasure/BorelCantelli.lean,Mathlib/RingTheory/HahnSeries/Valuation.lean,Mathlib/RingTheory/Valuation/Archimedean.lean,Mathlib/RingTheory/Valuation/ValuationRing.lean,Mathlib/RingTheory/Valuation/ValuativeRel/Basic.lean,Mathlib/SetTheory/Cardinal/Aleph.lean,Mathlib/SetTheory/Cardinal/Order.lean,Mathlib/Topology/EMetricSpace/BoundedVariation.lean,Mathlib/Topology/MetricSpace/HolderNorm.lean,Mathlib/Topology/UnitInterval.lean |
35 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
chrisflav assignee:chrisflav |
1-65957 1 day ago |
1-65958 1 day ago |
4-74424 4 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
- [x] depends on: #28511
- [x] depends on: #29207
- [x] depends on: #31143
- [x] depends on: #31144
- [x] depends on: #32253
- [ ] depends on: #32254
- [ ] depends on: #32398
[](https://gitpod.io/from-referrer/)
|
toric
large-import
t-algebra
blocked-by-other-PR
WIP
label:t-algebra$ |
810/639 |
Mathlib/Algebra/MonoidAlgebra/Defs.lean,Mathlib/Algebra/MonoidAlgebra/Degree.lean,Mathlib/Algebra/MonoidAlgebra/Division.lean,Mathlib/Algebra/MonoidAlgebra/Ideal.lean,Mathlib/Algebra/MonoidAlgebra/Lift.lean,Mathlib/Algebra/MonoidAlgebra/MapDomain.lean,Mathlib/Algebra/MonoidAlgebra/Module.lean,Mathlib/Algebra/MonoidAlgebra/NoZeroDivisors.lean,Mathlib/Algebra/MonoidAlgebra/Opposite.lean,Mathlib/Algebra/MonoidAlgebra/Support.lean,Mathlib/RingTheory/Finiteness/Finsupp.lean |
11 |
43 |
['JovanGerb', 'YaelDillies', 'alreadydone', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
1-61451 1 day ago |
3-1434 3 days ago |
36-61320 36 days |
| 30329 |
luigi-massacci author:luigi-massacci |
feat(Analysis/Distribution/TestFunction): integrating against a measure as a continuous linear map on test functions |
---
- [ ] depends on: #30004
- [ ] depends on: #32228
- [ ] depends on: #30327
- [x] depends on: #31806
- [x] depends on: #31533
- [x] depends on: #31470
- [ ] depends on: #30255
- [ ] depends on: #30253
- [ ] depends on: #30240
- [ ] depends on: #30239
- [x] depends on: #30236
- [x] depends on: #30202
- [x] depends on: #30201
- [x] depends on: #30199
- [x] depends on: #30198
- [x] depends on: #30197
[](https://gitpod.io/from-referrer/)
|
merge-conflict
blocked-by-other-PR
|
999/6 |
Mathlib.lean,Mathlib/Analysis/Distribution/ContDiffMapSupportedIn.lean,Mathlib/Analysis/Distribution/TestFunction.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/Data/Set/Function.lean,Mathlib/MeasureTheory/Integral/BoundedContinuousFunction.lean,Mathlib/MeasureTheory/Integral/TestAgainst.lean |
7 |
4 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
1-49758 1 day ago |
54-43681 1 month ago* |
0-1767 29 minutes* |
| 32147 |
EtienneC30 author:EtienneC30 |
feat: independence of Gaussian random variables |
Prove some results linking Gaussian random variables and independence. If `(X, Y)` is Gaussian, then `X` and `Y` are independent if their covariance is zero. Prove many versions of this theorem in different settings: in Banach spaces, Hilbert spaces, and for families of real random variables.
Also prove that independent Gaussian random variables are jointly Gaussian.
---
- [ ] depends on: #32144
- [ ] depends on: #30921
- [x] depends on: #32234
- [x] depends on: #32249
[](https://gitpod.io/from-referrer/)
|
brownian
t-measure-probability
blocked-by-other-PR
|
909/0 |
Mathlib.lean,Mathlib/Probability/Distributions/Gaussian/CharFun.lean,Mathlib/Probability/Distributions/Gaussian/HasGaussianLaw/Basic.lean,Mathlib/Probability/Distributions/Gaussian/HasGaussianLaw/Def.lean,Mathlib/Probability/Distributions/Gaussian/HasGaussianLaw/Independence.lean,Mathlib/Probability/Moments/CovarianceBilinDual.lean |
6 |
n/a |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
1-45262 1 day ago |
unknown |
unknown |
| 32330 |
ADedecker author:ADedecker |
feat: postcomposition by a CLM as a CLM on test functions |
---
- [ ] depends on: #32368
- [ ] depends on: #30239
[](https://gitpod.io/from-referrer/)
|
t-analysis
blocked-by-other-PR
|
99/3 |
Mathlib/Analysis/Distribution/ContDiffMapSupportedIn.lean,Mathlib/Analysis/Distribution/TestFunction.lean |
2 |
n/a |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
1-42574 1 day ago |
unknown |
unknown |
| 31809 |
ADedecker author:ADedecker |
feat: differentiation of test function as a CLM |
Co-authored-by: @luigi-massacci
---
- [x] depends on: #31806
- [ ] depends on: #30240
[](https://gitpod.io/from-referrer/)
|
t-analysis
blocked-by-other-PR
|
419/5 |
Mathlib/Analysis/Distribution/ContDiffMapSupportedIn.lean,Mathlib/Analysis/Distribution/TestFunction.lean |
2 |
n/a |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
1-41040 1 day ago |
unknown |
unknown |
| 32211 |
ADedecker author:ADedecker |
feat: inclusion from `ContDiffMapSupportedIn` to `TestFunction` is a topological embedding |
---
- [ ] depends on: #32210
- [x] depends on: #31806
[](https://gitpod.io/from-referrer/)
|
t-analysis
merge-conflict
blocked-by-other-PR
|
197/2 |
Mathlib/Analysis/Distribution/TestFunction.lean,Mathlib/Topology/UniformSpace/UniformEmbedding.lean |
2 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
1-39567 1 day ago |
3-68158 3 days ago |
0-2371 39 minutes |
| 32269 |
EtienneC30 author:EtienneC30 |
feat: introduce Gaussian processes |
Define Gaussian processes as stochastic processes whose finite dimensional distributions are Gaussian.
---
- [ ] depends on: #32144
- [x] depends on: #32274
[](https://gitpod.io/from-referrer/)
|
brownian
t-measure-probability
blocked-by-other-PR
|
481/0 |
Mathlib.lean,Mathlib/Probability/Distributions/Gaussian/HasGaussianLaw/Basic.lean,Mathlib/Probability/Distributions/Gaussian/HasGaussianLaw/Def.lean,Mathlib/Probability/Distributions/Gaussian/IsGaussianProcess/Basic.lean,Mathlib/Probability/Distributions/Gaussian/IsGaussianProcess/Def.lean |
5 |
n/a |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
1-38827 1 day ago |
unknown |
unknown |
| 32334 |
EtienneC30 author:EtienneC30 |
feat: independence of Gaussian processes |
Prove different versions of the following statement: if some stochastic processes are jointly Gaussian, then they are independent if their marginals are uncorrelated.
---
- [ ] depends on: #32147
- [ ] depends on: #32269
[](https://gitpod.io/from-referrer/)
|
brownian
t-measure-probability
blocked-by-other-PR
|
1291/0 |
Mathlib.lean,Mathlib/Probability/Distributions/Gaussian/CharFun.lean,Mathlib/Probability/Distributions/Gaussian/HasGaussianLaw/Basic.lean,Mathlib/Probability/Distributions/Gaussian/HasGaussianLaw/Def.lean,Mathlib/Probability/Distributions/Gaussian/HasGaussianLaw/Independence.lean,Mathlib/Probability/Distributions/Gaussian/IsGaussianProcess/Basic.lean,Mathlib/Probability/Distributions/Gaussian/IsGaussianProcess/Def.lean,Mathlib/Probability/Distributions/Gaussian/IsGaussianProcess/Independence.lean,Mathlib/Probability/Moments/CovarianceBilinDual.lean |
9 |
n/a |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
1-38740 1 day ago |
unknown |
unknown |
| 31795 |
thorimur author:thorimur |
feat: turn on `unusedFintypeInType` linter |
---
- [ ] depends on: #31794
- [x] depends on: #31747
[](https://gitpod.io/from-referrer/)
|
blocked-by-other-PR |
387/90 |
Mathlib/Analysis/Calculus/Deriv/Pi.lean,Mathlib/Analysis/Calculus/FDeriv/CompCLM.lean,Mathlib/Analysis/Calculus/FDeriv/Prod.lean,Mathlib/Analysis/Calculus/FDeriv/WithLp.lean,Mathlib/Analysis/InnerProductSpace/Calculus.lean,Mathlib/Analysis/SpecialFunctions/PolarCoord.lean,Mathlib/Combinatorics/SimpleGraph/Matching.lean,Mathlib/Data/Fintype/EquivFin.lean,Mathlib/Data/Fintype/Quotient.lean,Mathlib/GroupTheory/Perm/Cycle/Type.lean,Mathlib/Init.lean,Mathlib/MeasureTheory/Measure/HasOuterApproxClosedProd.lean,Mathlib/NumberTheory/JacobiSum/Basic.lean,Mathlib/Probability/Independence/BoundedContinuousFunction.lean,Mathlib/RepresentationTheory/Homological/FiniteCyclic.lean,Mathlib/RingTheory/AdicCompletion/AsTensorProduct.lean,Mathlib/Tactic/Linter/UnusedInstancesInType.lean,MathlibTest/UnusedInstancesInType.lean |
18 |
5 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
1-36215 1 day ago |
1-42880 1 day ago |
0-0 0 seconds |
| 32410 |
callesonne author:callesonne |
feat(Bicategory/FunctorCategory/Pseudo): Add evaluation pseudofunctor |
Adding pseudofunctors `eval` and `evaluation`. WIP PR to access CI.
---
- [ ] depends on: #30926
[](https://gitpod.io/from-referrer/)
|
t-category-theory
blocked-by-other-PR
WIP
|
160/31 |
Mathlib.lean,Mathlib/CategoryTheory/Bicategory/Functor/Lax.lean,Mathlib/CategoryTheory/Bicategory/Functor/Oplax.lean,Mathlib/CategoryTheory/Bicategory/Functor/Pseudofunctor.lean,Mathlib/CategoryTheory/Bicategory/Functor/StrictlyUnitary.lean,Mathlib/CategoryTheory/Bicategory/FunctorBicategory/Oplax.lean,Mathlib/CategoryTheory/Bicategory/FunctorBicategory/Pseudo.lean,Mathlib/CategoryTheory/Bicategory/Modification/Pseudo.lean,Mathlib/CategoryTheory/Bicategory/NaturalTransformation/Oplax.lean,Mathlib/CategoryTheory/Bicategory/NaturalTransformation/Pseudo.lean,Mathlib/CategoryTheory/Products/Basic.lean |
11 |
n/a |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
1-28982 1 day ago |
unknown |
unknown |
| 29819 |
mcdoll author:mcdoll |
feat(Analysis/Distribution): tempered distributions |
---
This is mainly a tracking PR: Most features will be PR'd separately.
- [x] depends on: #29818
- [x] depends on: #29821
- [x] depends on: #29846
- [x] depends on: #29860
- [x] depends on: #30174
- [x] depends on: #30175
- [x] depends on: #30176
- [x] depends on: #30180
- [x] depends on: #30195
- [x] depends on: #31075
- [x] depends on: #31074
- [x] depends on: #29888
- [x] depends on: #31073
- [ ] depends on: #29948
- [x] depends on: #31076
- [x] depends on: #31079
- [x] depends on: #31112
- [x] depends on: #31115
- [x] depends on: #31114
- [x] depends on: #11496
- [x] depends on: #31085
- [x] depends on: #31577
- [x] depends on: #31756
- [ ] depends on: #31757
- [x] depends on: #31760
- [ ] depends on: #32297
- [x] depends on: #32084
- [ ] depends on: #31876
- [ ] depends on: #32411
- [ ] depends on: #32307
[](https://gitpod.io/from-referrer/)
|
t-analysis
merge-conflict
blocked-by-other-PR
WIP
|
2365/156 |
Mathlib.lean,Mathlib/Analysis/Calculus/ContDiff/Bounds.lean,Mathlib/Analysis/Distribution/DenseLp.lean,Mathlib/Analysis/Distribution/FourierMultiplier.lean,Mathlib/Analysis/Distribution/FourierSchwartz.lean,Mathlib/Analysis/Distribution/SchwartzSpace.lean,Mathlib/Analysis/Distribution/TemperedDistribution.lean,Mathlib/Analysis/Fourier/FourierTransform.lean,Mathlib/Analysis/Fourier/L2Space.lean,Mathlib/Analysis/Fourier/Notation.lean,Mathlib/Analysis/Fourier/PoissonSummation.lean,Mathlib/Analysis/InnerProductSpace/Extend.lean,Mathlib/Analysis/InnerProductSpace/LinearPMap.lean,Mathlib/Analysis/LocallyConvex/Bounded.lean,Mathlib/Analysis/LocallyConvex/PointwiseConvergence.lean,Mathlib/Analysis/Normed/Operator/Completeness.lean,Mathlib/Analysis/Normed/Operator/Extend.lean,Mathlib/Analysis/SpecialFunctions/Gaussian/FourierTransform.lean,Mathlib/MeasureTheory/Integral/SetToL1.lean,Mathlib/Topology/Algebra/Module/PointwiseConvergence.lean,Mathlib/Topology/Algebra/Module/StrongTopology.lean,Mathlib/Topology/UniformSpace/UniformConvergenceTopology.lean,docs/undergrad.yaml |
23 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
1-22867 1 day ago |
65-38998 2 months ago |
0-2 2 seconds |
| 30563 |
YaelDillies author:YaelDillies |
chore(Algebra): replace `NoZeroSMulDivisors` with `Module.IsTorsionFree` |
`NoZeroSMulDivisors R M` is mathematically wrong when `R` isn't a domain, so we replace it with the better definition `Module.IsTorsionFree R M`. In fact, it never holds in such case unless `M` is trivial.
Here's a proof that `NoZeroSMulDivisors R M` implies `NoZeroDivisors R`.
If `m : M` is non-zero and `r s : R` are such that `r * s = 0`, then `r • s • m = (r * s) • m = 0`, so by `NoZeroSMulDivisors` we get `r = 0 ∨ s = 0 ∨ m = 0`. But `m ≠ 0`, so `r = 0 ∨ s = 0`, as wanted.
This means that one can eagerly replace `NoZeroSMulDivisors R M` with `NoZeroDivisors R` + `Module.IsTorsionFree R M`. Doing so, some lemmas become vacuous and some instances redundant. We remove them.
Since `NoZeroDivisors R` is usually mathematically incorrect when `R` is a semiring, I in fact replace `NoZeroSMulDivisors R M` with `IsDomain R` + `Module.IsTorsionFree R M`.
---
- [x] depends on: #30614
- [x] depends on: #30628
- [ ] depends on: #30678
- [x] depends on: #30683
- [x] depends on: #30707
- [x] depends on: #30708
- [x] depends on: #30716
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebra
blocked-by-other-PR
WIP
label:t-algebra$ |
1134/1331 |
Mathlib/Algebra/Algebra/Basic.lean,Mathlib/Algebra/Algebra/NonUnitalSubalgebra.lean,Mathlib/Algebra/Algebra/Subalgebra/Basic.lean,Mathlib/Algebra/Algebra/Tower.lean,Mathlib/Algebra/AlgebraicCard.lean,Mathlib/Algebra/BigOperators/Finprod.lean,Mathlib/Algebra/Central/Basic.lean,Mathlib/Algebra/CharP/LinearMaps.lean,Mathlib/Algebra/Group/Submonoid/Defs.lean,Mathlib/Algebra/GroupWithZero/Action/Pointwise/Finset.lean,Mathlib/Algebra/GroupWithZero/Action/Pointwise/Set.lean,Mathlib/Algebra/GroupWithZero/NonZeroDivisors.lean,Mathlib/Algebra/GroupWithZero/Regular.lean,Mathlib/Algebra/Lie/Sl2.lean,Mathlib/Algebra/Lie/Submodule.lean,Mathlib/Algebra/Lie/TraceForm.lean,Mathlib/Algebra/Lie/Weights/Basic.lean,Mathlib/Algebra/Lie/Weights/Chain.lean,Mathlib/Algebra/Lie/Weights/Linear.lean,Mathlib/Algebra/Module/Basic.lean,Mathlib/Algebra/Module/Card.lean,Mathlib/Algebra/Module/Lattice.lean,Mathlib/Algebra/Module/LinearMap/Basic.lean,Mathlib/Algebra/Module/LinearMap/End.lean,Mathlib/Algebra/Module/LocalizedModule/Basic.lean,Mathlib/Algebra/Module/NatInt.lean,Mathlib/Algebra/Module/Submodule/Basic.lean,Mathlib/Algebra/Module/Submodule/Lattice.lean,Mathlib/Algebra/Module/Submodule/Union.lean,Mathlib/Algebra/Module/Torsion/Basic.lean,Mathlib/Algebra/Module/Torsion/Free.lean,Mathlib/Algebra/Module/TransferInstance.lean,Mathlib/Algebra/MonoidAlgebra/Module.lean,Mathlib/Algebra/MvPolynomial/Basic.lean,Mathlib/Algebra/NoZeroSMulDivisors/Basic.lean,Mathlib/Algebra/NoZeroSMulDivisors/Defs.lean,Mathlib/Algebra/NoZeroSMulDivisors/Pi.lean,Mathlib/Algebra/NoZeroSMulDivisors/Prod.lean,Mathlib/Algebra/Order/BigOperators/Expect.lean,Mathlib/Algebra/Order/Module/Defs.lean,Mathlib/Algebra/Order/Module/Field.lean,Mathlib/Algebra/Order/Star/Basic.lean,Mathlib/Algebra/Polynomial/Basic.lean,Mathlib/Algebra/Polynomial/Degree/Domain.lean,Mathlib/Algebra/Polynomial/FieldDivision.lean,Mathlib/Algebra/Polynomial/Module/FiniteDimensional.lean,Mathlib/Algebra/Polynomial/Roots.lean,Mathlib/Algebra/Polynomial/Sequence.lean,Mathlib/Algebra/QuadraticAlgebra/Defs.lean,Mathlib/Algebra/Quaternion.lean,Mathlib/Algebra/Ring/Action/Pointwise/Finset.lean,Mathlib/Algebra/Ring/Action/Pointwise/Set.lean,Mathlib/Algebra/Star/NonUnitalSubalgebra.lean,Mathlib/Analysis/Analytic/IsolatedZeros.lean,Mathlib/Analysis/Analytic/OfScalars.lean,Mathlib/Analysis/Convex/Between.lean,Mathlib/Analysis/Convex/Extreme.lean,Mathlib/Analysis/Convex/Segment.lean,Mathlib/Analysis/Convex/Strict.lean,Mathlib/Analysis/Normed/Module/Ball/Action.lean,Mathlib/Analysis/SpecificLimits/Normed.lean,Mathlib/Data/ENNReal/Action.lean,Mathlib/Data/Finsupp/SMul.lean,Mathlib/Data/Finsupp/Weight.lean,Mathlib/FieldTheory/IsAlgClosed/Basic.lean,Mathlib/FieldTheory/Minpoly/IsConjRoot.lean,Mathlib/FieldTheory/Minpoly/IsIntegrallyClosed.lean,Mathlib/FieldTheory/PurelyInseparable/Basic.lean,Mathlib/FieldTheory/SplittingField/Construction.lean,Mathlib/FieldTheory/Tower.lean,Mathlib/Geometry/Euclidean/Triangle.lean,Mathlib/GroupTheory/GroupAction/Basic.lean,Mathlib/GroupTheory/Torsion.lean,Mathlib/LinearAlgebra/AffineSpace/AffineMap.lean,Mathlib/LinearAlgebra/AffineSpace/AffineSubspace/Basic.lean,Mathlib/LinearAlgebra/AffineSpace/Pointwise.lean,Mathlib/LinearAlgebra/AffineSpace/Slope.lean,Mathlib/LinearAlgebra/Alternating/Basic.lean,Mathlib/LinearAlgebra/Basis/Basic.lean,Mathlib/LinearAlgebra/Basis/Submodule.lean,Mathlib/LinearAlgebra/BilinearForm/DualLattice.lean,Mathlib/LinearAlgebra/BilinearForm/Properties.lean,Mathlib/LinearAlgebra/BilinearMap.lean,Mathlib/LinearAlgebra/DFinsupp.lean,Mathlib/LinearAlgebra/Dimension/Constructions.lean,Mathlib/LinearAlgebra/Dimension/Finite.lean,Mathlib/LinearAlgebra/Dimension/RankNullity.lean,Mathlib/LinearAlgebra/Dual/Defs.lean,Mathlib/LinearAlgebra/Eigenspace/Basic.lean,Mathlib/LinearAlgebra/Eigenspace/Matrix.lean,Mathlib/LinearAlgebra/Eigenspace/Minpoly.lean,Mathlib/LinearAlgebra/Eigenspace/Pi.lean,Mathlib/LinearAlgebra/Finsupp/VectorSpace.lean,Mathlib/LinearAlgebra/FreeModule/Basic.lean,Mathlib/LinearAlgebra/FreeModule/PID.lean,Mathlib/LinearAlgebra/LinearIndependent/Basic.lean,Mathlib/LinearAlgebra/LinearIndependent/Defs.lean,Mathlib/LinearAlgebra/LinearIndependent/Lemmas.lean,Mathlib/LinearAlgebra/LinearPMap.lean,Mathlib/LinearAlgebra/Matrix/Basis.lean |
174 |
24 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
0-86280 23 hours ago |
0-86301 23 hours ago |
0-119 1 minute |
| 32418 |
Thmoas-Guan author:Thmoas-Guan |
feat(RingTheory): Gorenstein local ring is Cohen--Macaulay local ring of type 1 |
In this PR, we formalized Theorem 18.1 of _Commutaive Ring Theory_ Matsumura.
This gives a full characterization of `Ext(k, R)` for Gorenstein local ring and implies that it is equivalent to Cohen--Macaulay local ring of type 1.
---
- [ ] depends on: #26245
- [ ] depends on: #30931
[](https://gitpod.io/from-referrer/)
|
merge-conflict
blocked-by-other-PR
|
6531/28 |
Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Baer.lean,Mathlib/Algebra/Category/ModuleCat/Ext/BaseChange.lean,Mathlib/Algebra/Category/ModuleCat/Ext/Finite.lean,Mathlib/Algebra/Category/ModuleCat/Ext/Ulift.lean,Mathlib/Algebra/Category/ModuleCat/InjectiveDimension.lean,Mathlib/Algebra/Category/ModuleCat/Localization.lean,Mathlib/Algebra/Category/ModuleCat/Ulift.lean,Mathlib/Algebra/Homology/DerivedCategory/ExactFunctor.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/Bijection.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/Map.lean,Mathlib/Algebra/Homology/DerivedCategory/ShortExact.lean,Mathlib/Algebra/Homology/HomotopyCategory.lean,Mathlib/Algebra/Homology/HomotopyCategory/Pretriangulated.lean,Mathlib/Algebra/Homology/HomotopyCategory/ShortExact.lean,Mathlib/Algebra/Module/Equiv/Basic.lean,Mathlib/Algebra/Module/FinitePresentation.lean,Mathlib/CategoryTheory/Abelian/Projective/Dimension.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/RingTheory/CohenMacaulay/Basic.lean,Mathlib/RingTheory/CohenMacaulay/Catenary.lean,Mathlib/RingTheory/Flat/IsBaseChange.lean,Mathlib/RingTheory/Gorenstein/CohenMacaulay.lean,Mathlib/RingTheory/Gorenstein/Defs.lean,Mathlib/RingTheory/Ideal/AssociatedPrime/Localization.lean,Mathlib/RingTheory/Regular/Category.lean,Mathlib/RingTheory/Regular/Depth.lean,Mathlib/RingTheory/Regular/InjectiveDimension.lean,Mathlib/RingTheory/Regular/Ischebeck.lean,Mathlib/RingTheory/Regular/ProjectiveDimension.lean |
30 |
n/a |
['mathlib4-dependent-issues-bot'] |
nobody |
0-84828 23 hours ago |
unknown |
unknown |
| 32294 |
jsm28 author:jsm28 |
feat(Geometry/Euclidean/Angle/Incenter): distance from second intersection with circumcircle |
Add the following lemma: given a triangle ABC, suppose an angle bisector from A through the incenter or excenter I meets the circumcircle again at X (including the case of an external bisector at A tangent to the circle, in which case X = A). Then XB = XI (= XC, by applying this lemma again). This is a standard configuration: https://en.wikipedia.org/wiki/Incenter%E2%80%93excenter_lemma
---
- [ ] depends on: #30981
- [ ] depends on: #30982
- [ ] depends on: #32019
- [ ] depends on: #32021
- [ ] depends on: #32023
- [ ] depends on: #32270
- [ ] depends on: #32290
[](https://gitpod.io/from-referrer/)
|
t-euclidean-geometry
blocked-by-other-PR
|
867/4 |
Mathlib.lean,Mathlib/Geometry/Euclidean/Altitude.lean,Mathlib/Geometry/Euclidean/Angle/Bisector.lean,Mathlib/Geometry/Euclidean/Angle/Incenter.lean,Mathlib/Geometry/Euclidean/Incenter.lean,Mathlib/Geometry/Euclidean/Projection.lean |
6 |
n/a |
['github-actions', 'jsm28', 'mathlib4-dependent-issues-bot', 'peakpoint'] |
nobody |
0-80660 22 hours ago |
unknown |
unknown |
| 32295 |
jsm28 author:jsm28 |
feat(Archive/Imo/Imo2024Q4): IMO 2024 Q4 |
Add a formalization of IMO 2024 problem 4, so completing the formalizations of all six IMO 2024 problems.
---
- [ ] depends on: #30981
- [ ] depends on: #30982
- [ ] depends on: #31057
- [ ] depends on: #31205
- [ ] depends on: #31452
- [ ] depends on: #31495
- [ ] depends on: #31733
- [ ] depends on: #31891
- [ ] depends on: #31892
- [ ] depends on: #31893
- [ ] depends on: #31979
- [ ] depends on: #31981
- [ ] depends on: #32004
- [ ] depends on: #32019
- [ ] depends on: #32021
- [ ] depends on: #32023
- [ ] depends on: #32259
- [ ] depends on: #32260
- [ ] depends on: #32270
- [ ] depends on: #32273
- [ ] depends on: #32278
- [ ] depends on: #32282
- [ ] depends on: #32290
- [ ] depends on: #32294
- [ ] depends on: #32296
[](https://gitpod.io/from-referrer/)
|
IMO
blocked-by-other-PR
|
2984/9 |
Archive.lean,Archive/Imo/Imo2024Q4.lean,Mathlib.lean,Mathlib/Analysis/Convex/Side.lean,Mathlib/Analysis/Convex/StrictCombination.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Angle.lean,Mathlib/Geometry/Euclidean/Altitude.lean,Mathlib/Geometry/Euclidean/Angle/Bisector.lean,Mathlib/Geometry/Euclidean/Angle/Incenter.lean,Mathlib/Geometry/Euclidean/Angle/Oriented/Affine.lean,Mathlib/Geometry/Euclidean/Angle/Sphere.lean,Mathlib/Geometry/Euclidean/Incenter.lean,Mathlib/Geometry/Euclidean/Projection.lean,Mathlib/Geometry/Euclidean/Sphere/OrthRadius.lean,Mathlib/Geometry/Euclidean/Sphere/PolePolar.lean,Mathlib/Geometry/Euclidean/Sphere/SecondInter.lean,Mathlib/Geometry/Euclidean/Sphere/Tangent.lean,Mathlib/LinearAlgebra/AffineSpace/Independent.lean |
18 |
n/a |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
0-80640 22 hours ago |
unknown |
unknown |
| 30817 |
joelriou author:joelriou |
feat(CategoryTheory): `κ`-continuous presheaves |
Given categories `C`, `D` and a regular cardinal `κ : Cardinal.{w}`, we define `isCardinalContinuous C D κ : ObjectProperty (C ⥤ D)` as the property of functors which preserves limits indexed by categories `J` such that `HasCardinalLT (Arrow J) κ`.
When `C : Type w` is a small category, we show that `κ`-continuous functors `Cᵒᵖ ⥤ Type w` are exactly the objects that are local with respect to a suitable `w`-small family of morphisms.
DRAFT
Note: definitions in `ObjectProperty.FunctorCategory.Limits` are duplicates of definitions in `ObjectProperty.FunctorCategory.PreservesLimits`.
---
- [x] depends on: #30168
- [x] depends on: #30160
- [x] depends on: #29881
- [x] depends on: #29854
[](https://gitpod.io/from-referrer/)
|
t-category-theory
blocked-by-other-PR
WIP
|
431/0 |
Mathlib.lean,Mathlib/CategoryTheory/Limits/Types/Limits.lean,Mathlib/CategoryTheory/MorphismProperty/Basic.lean,Mathlib/CategoryTheory/MorphismProperty/IsSmall.lean,Mathlib/CategoryTheory/ObjectProperty/FunctorCategory/Limits.lean,Mathlib/CategoryTheory/ObjectProperty/FunctorCategory/Presheaf.lean,Mathlib/CategoryTheory/ObjectProperty/Local.lean,Mathlib/CategoryTheory/Presentable/Continuous.lean |
8 |
8 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
0-79994 22 hours ago |
9-75811 9 days ago |
0-1 1 second |
| 30847 |
joelriou author:joelriou |
feat(CategoryTheory/Presentable): the representation theorem |
If `C` is an essentially `w`-small category, then the category of `κ`-continuous functors `Cᵒᵖ ⥤ Type w` is locally `κ`-presentable, and any locally `κ`-presentable category is equivalent to such a category. In particular, we show that a locally `κ`-presentable category has limits.
This is a draft...
---
- [ ] depends on: #32423
- [ ] depends on: #32424
- [ ] depends on: #32034
- [ ] depends on: #31137
- [ ] depends on: #30817
- [x] depends on: #30795
- [ ] depends on: #30755
- [ ] depends on: #30731
- [ ] depends on: #30554
- [ ] depends on: #30533
- [ ] depends on: #30513
- [x] depends on: #30509
- [x] depends on: #30507
- [x] depends on: #30492
- [x] depends on: #30464
- [x] depends on: #30459
- [x] depends on: #30269
- [ ] depends on: #30247
- [ ] depends on: #30241
- [x] depends on: #30168
- [x] depends on: #30160
- [x] depends on: #29881
- [x] depends on: #29854
- [x] depends on: #29565
- [x] depends on: #29543
- [x] depends on: #29519
[](https://gitpod.io/from-referrer/)
|
t-category-theory
merge-conflict
blocked-by-other-PR
WIP
|
2137/27 |
Mathlib.lean,Mathlib/CategoryTheory/Adjunction/Basic.lean,Mathlib/CategoryTheory/EssentiallySmall.lean,Mathlib/CategoryTheory/Functor/KanExtension/Dense.lean,Mathlib/CategoryTheory/Generator/Basic.lean,Mathlib/CategoryTheory/Generator/Type.lean,Mathlib/CategoryTheory/Limits/HasLimits.lean,Mathlib/CategoryTheory/Limits/Shapes/Multiequalizer.lean,Mathlib/CategoryTheory/Limits/Types/Limits.lean,Mathlib/CategoryTheory/MorphismProperty/Basic.lean,Mathlib/CategoryTheory/MorphismProperty/IsSmall.lean,Mathlib/CategoryTheory/ObjectProperty/Basic.lean,Mathlib/CategoryTheory/ObjectProperty/ClosedUnderIsomorphisms.lean,Mathlib/CategoryTheory/ObjectProperty/ColimitsCardinalClosure.lean,Mathlib/CategoryTheory/ObjectProperty/ColimitsOfShape.lean,Mathlib/CategoryTheory/ObjectProperty/CompleteLattice.lean,Mathlib/CategoryTheory/ObjectProperty/Equivalence.lean,Mathlib/CategoryTheory/ObjectProperty/FunctorCategory/Limits.lean,Mathlib/CategoryTheory/ObjectProperty/FunctorCategory/Presheaf.lean,Mathlib/CategoryTheory/ObjectProperty/LimitsOfShape.lean,Mathlib/CategoryTheory/ObjectProperty/Local.lean,Mathlib/CategoryTheory/ObjectProperty/Small.lean,Mathlib/CategoryTheory/Presentable/Adjunction.lean,Mathlib/CategoryTheory/Presentable/Basic.lean,Mathlib/CategoryTheory/Presentable/Continuous.lean,Mathlib/CategoryTheory/Presentable/Dense.lean,Mathlib/CategoryTheory/Presentable/EssentiallyLarge.lean,Mathlib/CategoryTheory/Presentable/Limits.lean,Mathlib/CategoryTheory/Presentable/LocallyPresentable.lean,Mathlib/CategoryTheory/Presentable/OrthogonalReflection.lean,Mathlib/CategoryTheory/Presentable/Presheaf.lean,Mathlib/CategoryTheory/Presentable/Representation.lean,Mathlib/CategoryTheory/Presentable/StrongGenerator.lean,Mathlib/CategoryTheory/Presentable/Type.lean,Mathlib/CategoryTheory/Yoneda.lean |
35 |
n/a |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
0-76973 21 hours ago |
unknown |
unknown |
| 30247 |
joelriou author:joelriou |
feat(CategoryTheory): categories of presheaves are locally presentable |
If `C` is a `w`-small category and `A` is locally `κ`-presentable, then the category `Cᵒᵖ ⥤ Type w` is locally `κ`-presentable; in particular, the category of presheaves of types on a small category is locally (finitely) presentable. (Currently, we formalise this under the additional assumption that `A` has pullbacks. This assumption shall be removed in the future as a locally presentable category is complete.)
---
- [ ] depends on: #30459
- [ ] depends on: #30241
- [ ] depends on: #30168
- [x] depends on: #29851
- [x] depends on: #29881
- [x] depends on: #29903
- [x] depends on: #29854
- [x] depends on: #30160
- [ ] depends on: #29565
- [x] depends on: #29556
- [x] depends on: #29519
- [x] depends on: #29518
- [x] depends on: #29543
[](https://gitpod.io/from-referrer/)
|
t-category-theory
blocked-by-other-PR
WIP
|
945/87 |
Mathlib.lean,Mathlib/CategoryTheory/EssentiallySmall.lean,Mathlib/CategoryTheory/Functor/KanExtension/Dense.lean,Mathlib/CategoryTheory/Generator/Basic.lean,Mathlib/CategoryTheory/Generator/Type.lean,Mathlib/CategoryTheory/Limits/HasLimits.lean,Mathlib/CategoryTheory/ObjectProperty/Basic.lean,Mathlib/CategoryTheory/ObjectProperty/ClosedUnderIsomorphisms.lean,Mathlib/CategoryTheory/ObjectProperty/ColimitsCardinalClosure.lean,Mathlib/CategoryTheory/ObjectProperty/ColimitsOfShape.lean,Mathlib/CategoryTheory/ObjectProperty/CompleteLattice.lean,Mathlib/CategoryTheory/ObjectProperty/Equivalence.lean,Mathlib/CategoryTheory/ObjectProperty/Small.lean,Mathlib/CategoryTheory/Presentable/Basic.lean,Mathlib/CategoryTheory/Presentable/CardinalFilteredPresentation.lean,Mathlib/CategoryTheory/Presentable/Limits.lean,Mathlib/CategoryTheory/Presentable/LocallyPresentable.lean,Mathlib/CategoryTheory/Presentable/Presheaf.lean,Mathlib/CategoryTheory/Presentable/StrongGenerator.lean,Mathlib/CategoryTheory/Presentable/Type.lean,Mathlib/CategoryTheory/SmallRepresentatives.lean |
21 |
5 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
0-74754 20 hours ago |
26-34889 26 days ago |
0-46 46 seconds |
| 31187 |
loefflerd author:loefflerd |
feat(NumberTheory/LSeries): Define the L-series of a modular form |
Define the L-function of a modular form (showing it is meromorphic on C and agrees with the naive Dirichlet series for `re s` large).
---
- [ ] depends on: #30089 |
t-number-theory
blocked-by-other-PR
WIP
|
616/26 |
Mathlib.lean,Mathlib/NumberTheory/LSeries/AbstractFuncEq.lean,Mathlib/NumberTheory/LSeries/HurwitzZetaOdd.lean,Mathlib/NumberTheory/ModularForms/Bounds.lean,Mathlib/NumberTheory/ModularForms/LFunction.lean,Mathlib/NumberTheory/ModularForms/QExpansion.lean |
6 |
n/a |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
0-73356 20 hours ago |
unknown |
unknown |
| 30799 |
YaelDillies author:YaelDillies |
refactor: unify the two versions of `pow_eq_one_iff` |
One version is about torsion-free monoids, the other one about linearly ordered monoids. I argue that all linearly ordered monoids of interest are torsion-free, and therefore the correct lemma to keep is the former.
[Zulip](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Should.20linear.20ordered.20comm.20monoids.20with.20zero.20be.20torsion-free)
---
- [x] depends on: #30680
- [x] depends on: #31024
- [x] depends on: #31025
- [x] depends on: #31026
- [x] depends on: #31027
- [x] depends on: #31283
- [ ] depends on: #31749
[](https://gitpod.io/from-referrer/)
|
file-removed
large-import
t-algebra
blocked-by-other-PR
label:t-algebra$ |
301/440 |
Counterexamples.lean,Counterexamples/LinearOrderWithPosMulPosEqZero.lean,Mathlib/Algebra/Group/Torsion.lean,Mathlib/Algebra/GroupWithZero/Torsion.lean,Mathlib/Algebra/Order/AddGroupWithTop.lean,Mathlib/Algebra/Order/Field/Canonical.lean,Mathlib/Algebra/Order/GroupWithZero/Canonical.lean,Mathlib/Algebra/Order/Monoid/Unbundled/Pow.lean,Mathlib/Algebra/Order/Nonneg/Ring.lean,Mathlib/Algebra/Order/PUnit.lean,Mathlib/Algebra/Order/Ring/Archimedean.lean,Mathlib/Algebra/Order/Ring/Basic.lean,Mathlib/Algebra/Order/Ring/Nat.lean,Mathlib/Algebra/Ring/NonZeroDivisors.lean,Mathlib/Algebra/Ring/Torsion.lean,Mathlib/Data/ENNReal/Basic.lean,Mathlib/Data/ENNReal/Real.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/Data/EReal/Operations.lean,Mathlib/Data/Nat/PartENat.lean,Mathlib/Data/Nat/Prime/Pow.lean,Mathlib/FieldTheory/Finite/GaloisField.lean,Mathlib/LinearAlgebra/Dimension/Finite.lean,Mathlib/MeasureTheory/Function/ConditionalExpectation/Real.lean,Mathlib/MeasureTheory/Function/ConvergenceInMeasure.lean,Mathlib/MeasureTheory/Integral/Bochner/Basic.lean,Mathlib/MeasureTheory/Integral/Bochner/Set.lean,Mathlib/MeasureTheory/Integral/Lebesgue/Basic.lean,Mathlib/MeasureTheory/Measure/Decomposition/Exhaustion.lean,Mathlib/MeasureTheory/Measure/Doubling.lean,Mathlib/MeasureTheory/Measure/EverywherePos.lean,Mathlib/MeasureTheory/Measure/LevyProkhorovMetric.lean,Mathlib/MeasureTheory/Measure/TightNormed.lean,Mathlib/MeasureTheory/OuterMeasure/BorelCantelli.lean,Mathlib/NumberTheory/ArithmeticFunction/Moebius.lean,Mathlib/RingTheory/HahnSeries/Valuation.lean,Mathlib/RingTheory/Valuation/Archimedean.lean,Mathlib/RingTheory/Valuation/Basic.lean,Mathlib/RingTheory/Valuation/ValuationRing.lean,Mathlib/RingTheory/Valuation/ValuativeRel/Basic.lean,Mathlib/RingTheory/ZMod/UnitsCyclic.lean,Mathlib/SetTheory/Cardinal/Aleph.lean,Mathlib/SetTheory/Cardinal/Order.lean,Mathlib/Topology/EMetricSpace/BoundedVariation.lean,Mathlib/Topology/MetricSpace/HolderNorm.lean,Mathlib/Topology/UnitInterval.lean |
46 |
13 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
0-72881 20 hours ago |
0-72903 20 hours ago |
0-10164 2 hours |
| 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
|
168/0 |
Mathlib.lean,Mathlib/RingTheory/RegularLocalRing/Defs.lean,Mathlib/RingTheory/RegularLocalRing/RegularRing/Basic.lean |
3 |
5 |
['Thmoas-Guan', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
0-68497 19 hours ago |
0-68497 19 hours ago |
0-153 2 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
merge-conflict
blocked-by-other-PR
|
3547/28 |
Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Baer.lean,Mathlib/Algebra/Category/ModuleCat/Ext/Finite.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/RingTheory/CohenMacaulay/Basic.lean,Mathlib/RingTheory/CohenMacaulay/Maximal.lean,Mathlib/RingTheory/GlobalDimension.lean,Mathlib/RingTheory/Ideal/AssociatedPrime/Localization.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 |
15 |
n/a |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
0-62447 17 hours ago |
unknown |
unknown |
| 29699 |
Thmoas-Guan author:Thmoas-Guan |
feat(Algebra/RingTheory): global dimension of regular ring |
In this PR, we proved that the global (homological dimension) of regular ring is equal to its krull dimension.
---
- [ ] depends on: #28684
- [ ] depends on: #31999
- [ ] depends on: #29534
[](https://gitpod.io/from-referrer/)
|
large-import
merge-conflict
blocked-by-other-PR
|
4079/28 |
Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Baer.lean,Mathlib/Algebra/Category/ModuleCat/Ext/Finite.lean,Mathlib/Algebra/Category/ModuleCat/Localization.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/RingTheory/CohenMacaulay/Basic.lean,Mathlib/RingTheory/CohenMacaulay/Maximal.lean,Mathlib/RingTheory/GlobalDimension.lean,Mathlib/RingTheory/Ideal/AssociatedPrime/Localization.lean,Mathlib/RingTheory/LocalProperties/ProjectiveDimension.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/RegularLocalRing/RegularRing/Basic.lean,Mathlib/RingTheory/RegularLocalRing/RegularRing/GlobalDimension.lean |
19 |
n/a |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
0-62446 17 hours ago |
unknown |
unknown |
| 29703 |
Thmoas-Guan author:Thmoas-Guan |
feat(Algebra/RingTheory): Hilbert's Syzygy theorem (projective version) |
In this PR, we proved for field `k`, `MvPolynomial (Fin n) k` has global dimension `n`.
---
- [ ] depends on: #29701
- [ ] depends on: #29699
[](https://gitpod.io/from-referrer/)
|
large-import
merge-conflict
blocked-by-other-PR
|
4335/28 |
Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Baer.lean,Mathlib/Algebra/Category/ModuleCat/Ext/Finite.lean,Mathlib/Algebra/Category/ModuleCat/Localization.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/RingTheory/CohenMacaulay/Basic.lean,Mathlib/RingTheory/CohenMacaulay/Maximal.lean,Mathlib/RingTheory/GlobalDimension.lean,Mathlib/RingTheory/Ideal/AssociatedPrime/Localization.lean,Mathlib/RingTheory/LocalProperties/ProjectiveDimension.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/RegularLocalRing/RegularRing/Basic.lean,Mathlib/RingTheory/RegularLocalRing/RegularRing/GlobalDimension.lean,Mathlib/RingTheory/RegularLocalRing/RegularRing/Polynomial.lean,Mathlib/RingTheory/RegularLocalRing/RegularRing/Syzygy.lean |
21 |
n/a |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
0-62444 17 hours ago |
unknown |
unknown |
| 29796 |
Thmoas-Guan author:Thmoas-Guan |
feat(RingTheory): regular of finite global dimension |
In this PR, we proved the other half of Auslander-Buchsbaum-Serre criterion, which states that a local ring is regular if it has finite global dimension, with results in #29557, we can obtain the full theorem. More APIs would be developed based on the two.
---
- [ ] depends on: #26215
- [ ] depends on: #26217
- [ ] depends on: #29558
- [ ] depends on: #28683
[](https://gitpod.io/from-referrer/)
|
large-import
merge-conflict
blocked-by-other-PR
|
3027/28 |
Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Baer.lean,Mathlib/Algebra/Category/ModuleCat/Ext/Finite.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/RingTheory/GlobalDimension.lean,Mathlib/RingTheory/Ideal/AssociatedPrime/Localization.lean,Mathlib/RingTheory/Regular/AuslanderBuchsbaum.lean,Mathlib/RingTheory/Regular/Category.lean,Mathlib/RingTheory/Regular/Depth.lean,Mathlib/RingTheory/Regular/Ischebeck.lean,Mathlib/RingTheory/RegularLocalRing/AuslanderBuchsbaumSerre.lean,Mathlib/RingTheory/RegularLocalRing/Basic.lean,Mathlib/RingTheory/RegularLocalRing/Defs.lean |
13 |
n/a |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
0-62443 17 hours ago |
unknown |
unknown |
| 29802 |
Thmoas-Guan author:Thmoas-Guan |
feat(Algebra/RingTheory): Auslander–Buchsbaum–Serre criterion and its corollaries |
In this PR, we proved that:
1: The full version of Auslander–Buchsbaum–Serre criterion
2: Localization of regular local ring is regular
3: Global dimension finite implies regular (doesn't need local)
4: Regular ring only need to be verified at maximal ideals.
---
- [ ] depends on: #29534
- [ ] depends on: #29699
[](https://gitpod.io/from-referrer/)
|
large-import
merge-conflict
blocked-by-other-PR
|
4890/28 |
Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Baer.lean,Mathlib/Algebra/Category/ModuleCat/Ext/Finite.lean,Mathlib/Algebra/Category/ModuleCat/Localization.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/RingTheory/CohenMacaulay/Basic.lean,Mathlib/RingTheory/CohenMacaulay/Maximal.lean,Mathlib/RingTheory/GlobalDimension.lean,Mathlib/RingTheory/Ideal/AssociatedPrime/Localization.lean,Mathlib/RingTheory/LocalProperties/ProjectiveDimension.lean,Mathlib/RingTheory/Regular/AuslanderBuchsbaum.lean,Mathlib/RingTheory/Regular/Category.lean,Mathlib/RingTheory/Regular/Depth.lean,Mathlib/RingTheory/Regular/Ischebeck.lean,Mathlib/RingTheory/RegularLocalRing/AuslanderBuchsbaumSerre.lean,Mathlib/RingTheory/RegularLocalRing/Basic.lean,Mathlib/RingTheory/RegularLocalRing/Defs.lean,Mathlib/RingTheory/RegularLocalRing/GlobalDimension.lean,Mathlib/RingTheory/RegularLocalRing/Localization.lean,Mathlib/RingTheory/RegularLocalRing/RegularRing/Basic.lean,Mathlib/RingTheory/RegularLocalRing/RegularRing/GlobalDimension.lean,Mathlib/RingTheory/RegularLocalRing/RegularRing/Localization.lean |
22 |
n/a |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
0-62441 17 hours ago |
unknown |
unknown |
| 31644 |
Thmoas-Guan author:Thmoas-Guan |
feat(Algebra): projective dimension of quotient regular sequence |
In this PR, we proved that for finitely generated module over Noetherian local ring, quotient by regular sequence increase the projective dimension by exactly its length.
---
- [ ] depends on: #32081
[](https://gitpod.io/from-referrer/)
|
t-ring-theory
merge-conflict
awaiting-author
blocked-by-other-PR
|
381/0 |
Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Ext/Finite.lean,Mathlib/CategoryTheory/Abelian/Projective/Dimension.lean,Mathlib/RingTheory/Regular/ProjectiveDimension.lean |
4 |
27 |
['Thmoas-Guan', 'erdOne', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
0-62069 17 hours ago |
0-62071 17 hours ago |
0-24742 6 hours |
| 31768 |
Thmoas-Guan author:Thmoas-Guan |
feat(Homology): `Ext` commute with ulift functor |
In this PR, we proved that `Ext` commute with ulift functor in `ModuleCat`.
Further more, we provided compatibility with (semi-)linear equiv of general universe.
---
- [ ] depends on: #31697
- [ ] depends on: #31706
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-category-theory
merge-conflict
blocked-by-other-PR
label:t-algebra$ |
840/0 |
Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Ext/Ulift.lean,Mathlib/Algebra/Category/ModuleCat/Ulift.lean,Mathlib/Algebra/Homology/DerivedCategory/ExactFunctor.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/Bijection.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/Map.lean,Mathlib/Algebra/Homology/DerivedCategory/ShortExact.lean,Mathlib/Algebra/Homology/HomotopyCategory.lean,Mathlib/Algebra/Homology/HomotopyCategory/Pretriangulated.lean,Mathlib/Algebra/Homology/HomotopyCategory/ShortExact.lean |
10 |
4 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
0-62068 17 hours ago |
0-62069 17 hours ago |
0-2065 34 minutes |
| 31851 |
Thmoas-Guan author:Thmoas-Guan |
feat(Algebra/Homology): Injective dimension in linear equiv |
In this PR, we proved that injective dimension is preserved under (semi-) linear equiv for general universe level.
---
- [ ] depends on: #31768
[](https://gitpod.io/from-referrer/)
|
t-algebra
merge-conflict
blocked-by-other-PR
label:t-algebra$ |
1083/0 |
Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Baer.lean,Mathlib/Algebra/Category/ModuleCat/Ext/Ulift.lean,Mathlib/Algebra/Category/ModuleCat/InjectiveDimension.lean,Mathlib/Algebra/Category/ModuleCat/Ulift.lean,Mathlib/Algebra/Homology/DerivedCategory/ExactFunctor.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/Bijection.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/Map.lean,Mathlib/Algebra/Homology/DerivedCategory/ShortExact.lean,Mathlib/Algebra/Homology/HomotopyCategory.lean,Mathlib/Algebra/Homology/HomotopyCategory/Pretriangulated.lean,Mathlib/Algebra/Homology/HomotopyCategory/ShortExact.lean |
12 |
2 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
0-61552 17 hours ago |
14-58278 14 days ago |
0-8108 2 hours |
| 31884 |
Thmoas-Guan author:Thmoas-Guan |
feat(RingTheory): definition of Gorenstein local ring |
In this PR, we gave basic definition of Gorenstein local ring and Gorestein ring and prove that they are stable under ring equiv.
---
- [ ] depends on: #31851
[](https://gitpod.io/from-referrer/)
|
merge-conflict
blocked-by-other-PR
|
1170/0 |
Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Baer.lean,Mathlib/Algebra/Category/ModuleCat/Ext/Ulift.lean,Mathlib/Algebra/Category/ModuleCat/InjectiveDimension.lean,Mathlib/Algebra/Category/ModuleCat/Ulift.lean,Mathlib/Algebra/Homology/DerivedCategory/ExactFunctor.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/Bijection.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/Map.lean,Mathlib/Algebra/Homology/DerivedCategory/ShortExact.lean,Mathlib/Algebra/Homology/HomotopyCategory.lean,Mathlib/Algebra/Homology/HomotopyCategory/Pretriangulated.lean,Mathlib/Algebra/Homology/HomotopyCategory/ShortExact.lean,Mathlib/RingTheory/Gorenstein/Defs.lean |
13 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
0-61550 17 hours ago |
0-61551 17 hours ago |
0-2574 42 minutes |
| 32035 |
Thmoas-Guan author:Thmoas-Guan |
feat(RingTheory): localization of Gorenstein local ring |
In this PR, we proved that localization of Gorenstein local ring at prime is again Gorenstein.
---
- [ ] depends on: #31884
- [ ] depends on: #32033
[](https://gitpod.io/from-referrer/)
|
merge-conflict
blocked-by-other-PR
|
1832/0 |
Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Baer.lean,Mathlib/Algebra/Category/ModuleCat/Ext/Ulift.lean,Mathlib/Algebra/Category/ModuleCat/InjectiveDimension.lean,Mathlib/Algebra/Category/ModuleCat/Localization.lean,Mathlib/Algebra/Category/ModuleCat/Ulift.lean,Mathlib/Algebra/Homology/DerivedCategory/ExactFunctor.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/Bijection.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/Map.lean,Mathlib/Algebra/Homology/DerivedCategory/ShortExact.lean,Mathlib/Algebra/Homology/HomotopyCategory.lean,Mathlib/Algebra/Homology/HomotopyCategory/Pretriangulated.lean,Mathlib/Algebra/Homology/HomotopyCategory/ShortExact.lean,Mathlib/RingTheory/Gorenstein/Basic.lean,Mathlib/RingTheory/Gorenstein/Defs.lean,Mathlib/RingTheory/LocalProperties/Injective.lean,Mathlib/RingTheory/LocalProperties/InjectiveDimension.lean |
17 |
n/a |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
0-61548 17 hours ago |
unknown |
unknown |
| 32098 |
Thmoas-Guan author:Thmoas-Guan |
feat(RingTheory): injective dimension of quotSMulTop |
In this PR, we proved for finitely generated module `M` over noetherian ring `R`, if `x` in maximal ideal being both `R`-regular and `M`-regular, `injdim_R (M/xM) + 1 = injdim_{R/(x)} (M)`.
---
- [ ] depends on: #31046
- [ ] depends on: #32058
- [ ] depends on: #32081
[](https://gitpod.io/from-referrer/)
|
merge-conflict
blocked-by-other-PR
|
1210/0 |
Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Baer.lean,Mathlib/Algebra/Category/ModuleCat/Ext/Finite.lean,Mathlib/Algebra/Homology/DerivedCategory/ExactFunctor.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/Map.lean,Mathlib/Algebra/Homology/DerivedCategory/ShortExact.lean,Mathlib/Algebra/Homology/HomotopyCategory.lean,Mathlib/Algebra/Homology/HomotopyCategory/Pretriangulated.lean,Mathlib/Algebra/Homology/HomotopyCategory/ShortExact.lean,Mathlib/RingTheory/Regular/InjectiveDimension.lean |
10 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
0-61544 17 hours ago |
0-61546 17 hours ago |
0-2059 34 minutes |
| 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$ |
662/6 |
Mathlib/RingTheory/Regular/Category.lean,Mathlib/RingTheory/Regular/Depth.lean |
2 |
n/a |
['Thmoas-Guan', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
0-60321 16 hours ago |
unknown |
unknown |
| 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$ |
964/6 |
Mathlib/RingTheory/Regular/Category.lean,Mathlib/RingTheory/Regular/Depth.lean |
2 |
n/a |
['Thmoas-Guan', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
0-60219 16 hours ago |
unknown |
unknown |
| 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
|
473/0 |
Mathlib.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/RingTheory/RegularLocalRing/Basic.lean,Mathlib/RingTheory/RegularLocalRing/Defs.lean |
4 |
5 |
['Thmoas-Guan', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
0-60081 16 hours ago |
15-1335 15 days ago |
0-111 1 minute |
| 32305 |
faenuccio author:faenuccio |
feat: define Weak Derivatives |
Nothing to see yet.
---
- [ ] depends on: #32250
[](https://gitpod.io/from-referrer/)
|
large-import
t-analysis
merge-conflict
blocked-by-other-PR
WIP
|
1795/5 |
Mathlib.lean,Mathlib/Analysis/Distribution/ContDiffMapSupportedIn.lean,Mathlib/Analysis/Distribution/Distribution.lean,Mathlib/Analysis/Distribution/TestFunction.lean,Mathlib/Analysis/Distribution/WeakDeriv.lean,Mathlib/Analysis/FunctionalSpaces/Sobolev/Basic.lean,Mathlib/MeasureTheory/Function/LocallyIntegrable.lean |
7 |
n/a |
['ADedecker', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
0-58529 16 hours ago |
unknown |
unknown |
| 30551 |
smmercuri author:smmercuri |
feat: dimension formulae for infinite places above |
---
- [x] depends on: #27978
- [x] depends on: #27974
- [ ] depends on: #29942
- [x] depends on: #29946
[](https://gitpod.io/from-referrer/)
|
merge-conflict
blocked-by-other-PR
WIP
|
613/7 |
Mathlib/Analysis/Normed/Field/WithAbs.lean,Mathlib/NumberTheory/NumberField/InfinitePlace/Completion.lean,Mathlib/NumberTheory/NumberField/InfinitePlace/Dimension.lean,Mathlib/NumberTheory/NumberField/InfinitePlace/Embeddings.lean,Mathlib/NumberTheory/NumberField/InfinitePlace/Ramification.lean |
5 |
5 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
0-39514 10 hours ago |
6-41640 6 days ago |
0-10 10 seconds |
| 31885 |
CoolRmal author:CoolRmal |
feat: Integrable if UI + convergence in measure |
---
- [ ] depends on: #31886
[](https://gitpod.io/from-referrer/)
|
brownian
t-measure-probability
blocked-by-other-PR
|
106/9 |
Mathlib/MeasureTheory/Function/ConvergenceInMeasure.lean,Mathlib/MeasureTheory/Function/UniformIntegrable.lean |
2 |
5 |
['EtienneC30', 'RemyDegenne', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
EtienneC30 assignee:EtienneC30 |
0-27212 7 hours ago |
0-33152 9 hours ago |
0-10728 2 hours |
| 32454 |
Hagb author:Hagb |
chore: simplify some proofs with `wlog!` |
This commit simplifies some proofs that used `wlog` and did things `push_neg`
does, with `wlog!` a new variant of `wlog`.
---
- [ ] depends on: #32453
[](https://gitpod.io/from-referrer/)
|
blocked-by-other-PR |
186/74 |
Counterexamples/AharoniKorman.lean,Mathlib/Algebra/CharP/Defs.lean,Mathlib/Algebra/Order/Field/Basic.lean,Mathlib/Algebra/Polynomial/RuleOfSigns.lean,Mathlib/Analysis/AbsoluteValue/Equivalence.lean,Mathlib/Analysis/Analytic/IsolatedZeros.lean,Mathlib/Analysis/Calculus/ContDiff/FaaDiBruno.lean,Mathlib/Analysis/Normed/Field/Basic.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Bounds.lean,Mathlib/CategoryTheory/Limits/Shapes/Countable.lean,Mathlib/Data/Set/Enumerate.lean,Mathlib/GroupTheory/ArchimedeanDensely.lean,Mathlib/GroupTheory/OreLocalization/Cardinality.lean,Mathlib/Logic/Godel/GodelBetaFunction.lean,Mathlib/MeasureTheory/Constructions/Polish/Basic.lean,Mathlib/Order/Fin/Basic.lean,Mathlib/Probability/Moments/IntegrableExpMul.lean,Mathlib/RingTheory/MvPolynomial/MonomialOrder.lean,Mathlib/Tactic/WLOG.lean,Mathlib/Topology/Algebra/Order/Group.lean,Mathlib/Topology/Algebra/Valued/LocallyCompact.lean,Mathlib/Topology/EMetricSpace/PairReduction.lean,Mathlib/Topology/MetricSpace/Ultra/Basic.lean,Mathlib/Topology/Order/LeftRightNhds.lean,MathlibTest/wlog.lean |
25 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot'] |
nobody |
0-12228 3 hours ago |
0-14418 3 hours ago |
0-1572 26 minutes |
| 32105 |
joelriou author:joelriou |
feat(CategoryTheory): computing Ext-groups using an injective resolution |
Given an injective resolution `R` of an object `Y` in an abelian category, we define a constructor for elements in `Ext X Y n` which takes as input "cocycles" given as morphisms `X ⟶ R.cocomplex.X n`, and we provide API for this definition.
When the dual construction for projective resolution will be done, it will be possible to remove the old `Ext` API.
DRAFT
---
- [ ] depends on: #32439
- [x] depends on: #32003
- [x] depends on: #32093
- [x] depends on: #32091
- [x] depends on: #32097
- [x] depends on: #31900
- [x] depends on: #31941
- [x] depends on: #31843
[](https://gitpod.io/from-referrer/)
|
large-import
t-category-theory
blocked-by-other-PR
WIP
|
626/6 |
Mathlib.lean,Mathlib/Algebra/Homology/DerivedCategory/Basic.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/Basic.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/TStructure.lean,Mathlib/Algebra/Homology/DerivedCategory/KInjective.lean,Mathlib/Algebra/Homology/DerivedCategory/SmallShiftedHom.lean,Mathlib/Algebra/Homology/DerivedCategory/TStructure.lean,Mathlib/Algebra/Homology/Embedding/IsSupported.lean,Mathlib/Algebra/Homology/HomotopyCategory/HomComplex.lean,Mathlib/Algebra/Homology/HomotopyCategory/HomComplexCohomology.lean,Mathlib/Algebra/Homology/HomotopyCategory/HomComplexSingle.lean,Mathlib/CategoryTheory/Abelian/Injective/Ext.lean,Mathlib/CategoryTheory/Abelian/Injective/Extend.lean,Mathlib/CategoryTheory/Localization/SmallShiftedHom.lean |
14 |
3 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
0-1646 27 minutes ago |
0-60690 16 hours ago |
0-817 13 minutes |
| 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
- [ ] depends on: #32316
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebra
blocked-by-other-PR
label:t-algebra$ |
1223/6 |
Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Ext/DimensionShifting.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/EnoughInjectives.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/EnoughProjectives.lean,Mathlib/RingTheory/Regular/AuslanderBuchsbaum.lean,Mathlib/RingTheory/Regular/Category.lean,Mathlib/RingTheory/Regular/Depth.lean |
7 |
n/a |
['Thmoas-Guan', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
0-1035 17 minutes ago |
unknown |
unknown |
| 32081 |
Thmoas-Guan author:Thmoas-Guan |
feat(RingTheory/Homology): `Ext` over Noetherian ring finitely generated |
In this PR, we proved that for `Ext` between finitely generated modules over Noetherian ring finitely generated.
---
- [ ] depends on: #32316
[](https://gitpod.io/from-referrer/)
|
t-algebra
t-category-theory
blocked-by-other-PR
label:t-algebra$ |
161/0 |
Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Ext/DimensionShifting.lean,Mathlib/Algebra/Category/ModuleCat/Ext/Finite.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/EnoughInjectives.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/EnoughProjectives.lean |
5 |
9 |
['Thmoas-Guan', 'dagurtomas', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
0-316 5 minutes ago |
0-60378 16 hours ago |
1-68433 1 day |
| 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.
---
- [x] 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$ |
2008/6 |
Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Ext/DimensionShifting.lean,Mathlib/Algebra/Category/ModuleCat/Ext/Finite.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/EnoughInjectives.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/EnoughProjectives.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/RingTheory/CohenMacaulay/Basic.lean,Mathlib/RingTheory/Regular/Category.lean,Mathlib/RingTheory/Regular/Depth.lean,Mathlib/RingTheory/Regular/Ischebeck.lean |
10 |
n/a |
['Thmoas-Guan', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
0-274 4 minutes 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$ |
2400/6 |
Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Ext/DimensionShifting.lean,Mathlib/Algebra/Category/ModuleCat/Ext/Finite.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/EnoughInjectives.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/EnoughProjectives.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/RingTheory/CohenMacaulay/Basic.lean,Mathlib/RingTheory/CohenMacaulay/Catenary.lean,Mathlib/RingTheory/Regular/Category.lean,Mathlib/RingTheory/Regular/Depth.lean,Mathlib/RingTheory/Regular/Ischebeck.lean |
11 |
n/a |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
0-273 4 minutes 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
- [ ] depends on: #32081
[](https://gitpod.io/from-referrer/)
|
large-import
t-algebra
blocked-by-other-PR
label:t-algebra$ |
1108/6 |
Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Ext/DimensionShifting.lean,Mathlib/Algebra/Category/ModuleCat/Ext/Finite.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/EnoughInjectives.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/EnoughProjectives.lean,Mathlib/RingTheory/Regular/Category.lean,Mathlib/RingTheory/Regular/Depth.lean,Mathlib/RingTheory/Regular/Ischebeck.lean |
8 |
n/a |
['Thmoas-Guan', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
0-273 4 minutes 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$ |
2584/6 |
Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Ext/DimensionShifting.lean,Mathlib/Algebra/Category/ModuleCat/Ext/Finite.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/EnoughInjectives.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/EnoughProjectives.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/RingTheory/CohenMacaulay/Basic.lean,Mathlib/RingTheory/CohenMacaulay/Catenary.lean,Mathlib/RingTheory/CohenMacaulay/Unmixed.lean,Mathlib/RingTheory/Regular/Category.lean,Mathlib/RingTheory/Regular/Depth.lean,Mathlib/RingTheory/Regular/Ischebeck.lean |
12 |
n/a |
['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
0-259 4 minutes ago |
unknown |
unknown |
| 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
|
3001/57 |
Mathlib.lean,Mathlib/Algebra/Category/Grp/Preadditive.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/Basic.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/Linear.lean,Mathlib/Algebra/Homology/DerivedCategory/Linear.lean,Mathlib/CategoryTheory/Shift/ShiftedHom.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 |
23 |
4 |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
0-248 4 minutes ago |
53-46226 1 month ago* |
0-88 1 minute* |
| 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
|
3166/6 |
Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Ext/DimensionShifting.lean,Mathlib/Algebra/Category/ModuleCat/Ext/Finite.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/EnoughInjectives.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/EnoughProjectives.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/RingTheory/CohenMacaulay/Basic.lean,Mathlib/RingTheory/CohenMacaulay/Maximal.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 |
15 |
n/a |
['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] |
nobody |
0-234 3 minutes ago |
unknown |
unknown |