Mathlib triage dashboard

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.

This dashboard was last updated on: January 15, 2026 at 09:42 UTC

Quick links: PR statistics | Not yet landed PRs | Review status | Stale unassigned PRs | Stale assigned PRs | Likely-spurious CI failures | Tech debt PRs | PRs blocked on a zulip discussion | PRs with just a merge conflict | Stale new contributor PRs | PRs not into master | PRs with an 'approved' review | All open PRs | Other lists of PRs

Overall statistics

Found 2009 open PRs overall. Among these PRs

Approved, not yet landed PRs

At the moment,

Review status

There are currently 255 PRs awaiting review. Among these,

On the other hand, 17 PRs are unassigned and have not seen a status change in a week, and 41 PRs are assigned, without recent review activity.

Stale unassigned PRs on the review queue

Number Author Title Description Labels +/- Modified files (first 100) 📝 💬 All users who commented or reviewed Assignee(s) Approval(s) Updated Last status change total time in review
33363 BoltonBailey
author:BoltonBailey
feat: add `empty_eq_image` simp lemmas Creates new simp lemmas `image_eq_empty`, similar to existing simp lemmas, but with the LHS equality reversed, so that simp can identify these when in this form. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data 7/0 Mathlib/Data/Finset/Image.lean,Mathlib/Data/Set/Image.lean 2 1 ['github-actions'] nobody none
17-38072
17 days ago
17-34732
17 days ago
17-34553
17 days
33481 NoneMore
author:NoneMore
feat(ModelTheory/Encoding): add `Countable` instances for (bounded) formulas in countable languages Prepare for the OTT proof. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-logic new-contributor 27/0 Mathlib/ModelTheory/Encoding.lean 1 1 ['github-actions'] nobody none
12-15014
12 days ago
12-14078
12 days ago
12-81800
12 days
33520 NoneMore
author:NoneMore
feat(ModelTheory/ElementarySubstructures): add a variant of Tarski-Vaught test taking sets as input There should exist an `ElementarySubstructure.copy` such that we can directly bundle the set itself instaed of its closure as an elementary substructure. The other direction depends on #33458. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-logic new-contributor 63/0 Mathlib/ModelTheory/ElementarySubstructures.lean 1 1 ['github-actions'] nobody none
11-68453
11 days ago
11-79856
11 days ago
11-79677
11 days
33475 BoltonBailey
author:BoltonBailey
feat(Logic/IsEmpty): add theorems relating surjectivity and emptiness In particular, this adds a lemma saying that with an empty domain, a function is surjective iff its range is empty, and various forms of this. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-logic 11/2 Mathlib/Logic/IsEmpty.lean 1 13 ['BoltonBailey', 'SnirBroshi', 'eric-wieser', 'github-actions'] nobody none
11-3215
11 days ago
10-85800
10 days ago
13-10412
13 days
33599 nielstron
author:nielstron
feat(Computability/ContextFreeGrammar): closure under union --- This PR picks up https://github.com/leanprover-community/mathlib4/pull/13514 and resolves the outstanding errors. - [ ] depends on #33592 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-computability new-contributor 506/0 Mathlib/Computability/ContextFreeGrammar.lean 1 1 ['github-actions'] nobody none
9-65132
9 days ago
9-71028
9 days ago
9-70849
9 days
33490 YaelDillies
author:YaelDillies
refactor(Data/Finsupp): remove `DecidableEq` argument from `curry` This is motivated by it spuriously requiring extra decidability assumptions in group cohomology. This partially reverts #24746. No motivation was given there for why computability was necessary. `Finsupp.curry` will be made computable again anyway once `Finsupp` is redefined to be `DFinsupp`. From ClassFieldTheory --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) CFT t-data 15/21 Mathlib/Data/Finsupp/Basic.lean,Mathlib/LinearAlgebra/Finsupp/Defs.lean,Mathlib/LinearAlgebra/Finsupp/LinearCombination.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/Basic.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/FiniteCyclic.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/Shapiro.lean,Mathlib/RepresentationTheory/Homological/Resolution.lean,Mathlib/RepresentationTheory/Rep.lean,Mathlib/RingTheory/AlgebraTower.lean 9 5 ['YaelDillies', 'eric-wieser', 'github-actions', 'tb65536'] nobody none
9-50006
9 days ago
11-79368
11 days ago
11-79189
11 days
33749 plp127
author:plp127
feat: `NNRat` is countable We provide an `Encodable NNRat` instance. As a consequence we also get the instance `Countable NNRat`. See also [Zulip](https://leanprover.zulipchat.com/#narrow/channel/113489-new-members/topic/NNRat.20not.20countable.3F/near/566916284) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data large-import 13/0 Mathlib/Data/Rat/Encodable.lean 1 4 ['eric-wieser', 'github-actions', 'grunweg', 'leanprover-radar'] nobody none
6-42530
6 days ago
6-39718
6 days ago
6-75554
6 days
33656 metakunt
author:metakunt
feat(Data/Nat/Choose): Add sum_range_multichoose t-data 11/0 Mathlib/Data/Nat/Choose/Sum.lean 1 6 ['eric-wieser', 'github-actions', 'metakunt'] nobody none
5-62099
5 days ago
9-7155
9 days ago
9-6976
9 days
33551 metakunt
author:metakunt
feat(Data/Nat/Factorization/PrimePow): Add Nat.nontrivial_primeFactors_of_two_le_of_not_isPrimePow t-data 6/0 Mathlib/Data/Nat/Factorization/PrimePow.lean 1 4 ['Ruben-VandeVelde', 'github-actions', 'metakunt'] nobody none
5-61620
5 days ago
5-61452
5 days ago
9-78323
9 days
33501 SnirBroshi
author:SnirBroshi
feat(Combinatorics/SimpleGraph/Finite): degrees for infinite graphs - Redefine degrees using `Set.ncard` to avoid `Fintype` and enable talking about degrees in infinite graphs. - Define `ENat` versions of `degree`/`minDegree`/`maxDegree` called `edegree`/`eminDegree`/`emaxDegree` respectively. - Remove `LocallyFinite` assumption from `IsRegularOfDegree`, and change it to use `edegree = k` instead of `degree = k` to retain the meaning of the case `k = 0`. --- The `e` prefix matches the existing `edist` and `ediam`. To make reviewing easier, this PR intentionally does not: - Add theorems about the new definitions - Reorder theorems to avoid `omit`s - Move theorems to a new `Degree.lean` file This is so that the diff shows the old/new versions side-by-side, and to avoid a bigger PR. Consequently a few proofs are a bit longer, but that'll be fixed after this PR by adding API lemmas for the new definitions (e.g. `edegree ≠ ⊤ → edegree = degree`). Regarding computability: If computability of degrees is useful, we can introduce a separate `findegree` in the future (similar to `neighborSet` vs `neighborFinset`), but I think degrees are a basic graph definition that should be defined for any `SimpleGraph`. As for theorems, such a `findegree` can use a lemma `findegree = degree` to access all the degree theorems, instead of duplicating everything to both versions. This PR was motivated by wanting to talk about infinite graphs with a finite max-degree. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-combinatorics 302/243 Archive/Wiedijk100Theorems/FriendshipGraphs.lean,Archive/Wiedijk100Theorems/Konigsberg.lean,Counterexamples/HeawoodUnitDistance.lean,Mathlib/Combinatorics/SimpleGraph/Acyclic.lean,Mathlib/Combinatorics/SimpleGraph/AdjMatrix.lean,Mathlib/Combinatorics/SimpleGraph/Bipartite.lean,Mathlib/Combinatorics/SimpleGraph/Circulant.lean,Mathlib/Combinatorics/SimpleGraph/Connectivity/Connected.lean,Mathlib/Combinatorics/SimpleGraph/DegreeSum.lean,Mathlib/Combinatorics/SimpleGraph/Extremal/Turan.lean,Mathlib/Combinatorics/SimpleGraph/Finite.lean,Mathlib/Combinatorics/SimpleGraph/FiveWheelLike.lean,Mathlib/Combinatorics/SimpleGraph/LapMatrix.lean,Mathlib/Combinatorics/SimpleGraph/Maps.lean,Mathlib/Combinatorics/SimpleGraph/Prod.lean,Mathlib/Combinatorics/SimpleGraph/StronglyRegular.lean,Mathlib/Combinatorics/SimpleGraph/Subgraph.lean,Mathlib/Combinatorics/SimpleGraph/Trails.lean,Mathlib/Data/Set/Card.lean,Mathlib/Data/Set/Insert.lean,Mathlib/Order/ConditionallyCompleteLattice/Finset.lean 21 1 ['github-actions'] nobody none
4-31153
4 days ago
11-62191
11 days ago
11-62012
11 days
33709 wangying11123
author:wangying11123
feat(Analysis/Convex/Between): Add wbtw_of_sameRay_vsub_left add wbtw_of_sameRay_vsub_left Main additions `wbtw_of_sameRay_vsub_left` if the vectors from a point x to points y and z lie on the same ray, then y is weakly between x and z, or z is weakly between x and y. new-contributor t-convex-geometry 24/0 Mathlib/Analysis/Convex/Between.lean 1 3 ['MichaelStollBayreuth', 'github-actions'] nobody none
3-54770
3 days ago
7-80089
7 days ago
7-79910
7 days
33254 SnirBroshi
author:SnirBroshi
feat(Data/Nat/Lattice): `¬BddAbove s → sSup s = 0` --- Note that it can also be proven `by simp [h]` after the `ConditionallyCompleteLinearOrderBot` instance below it. The theorem name matches the same theorems for other types: `Int.csSup_of_not_bdd_above`, `Real.sSup_of_not_bddAbove`, `NNReal.sSup_of_not_bddAbove`. Also renamed related `Int` theorems to conform to the naming conventions. [Zulip](https://leanprover.zulipchat.com/#narrow/channel/217875-Is-there-code-for-X.3F/topic/.60.C2.ACBddAbove.20s.20.E2.86.92.20sSup.20s.20.3D.200.60/with/565275221) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data 15/4 Mathlib/Data/Int/ConditionallyCompleteOrder.lean,Mathlib/Data/Nat/Lattice.lean 2 3 ['SnirBroshi', 'artie2000', 'github-actions', 'vihdzp'] nobody 2
3-53714
3 days ago
21-50060
21 days ago
21-69497
21 days
33845 bjornsolheim
author:bjornsolheim
feat(Analysis/Convex): barycenter of a standard simplex barycenter of a standard simplex --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis 26/0 Mathlib/Analysis/Convex/StdSimplex.lean 1 5 ['bjornsolheim', 'eric-wieser', 'github-actions'] nobody none
3-33331
3 days ago
3-31816
3 days ago
3-55344
3 days
33840 vihdzp
author:vihdzp
feat(SetTheory/Ordinal/CantorNormalForm): Evaluate a Finsupp as a CNF --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-set-theory 191/18 Mathlib/SetTheory/Ordinal/Arithmetic.lean,Mathlib/SetTheory/Ordinal/CantorNormalForm.lean 2 3 ['github-actions', 'plp127', 'vihdzp'] nobody none
3-32712
3 days ago
3-31761
3 days ago
3-36650
3 days
33860 DavidLedvinka
author:DavidLedvinka
feat(Probability): Add Cauchy distribution t-measure-probability 125/0 Mathlib.lean,Mathlib/Probability/Distributions/Cauchy.lean 2 1 ['github-actions'] nobody none
3-29733
3 days ago
3-28862
3 days ago
3-28683
3 days
33852 zcyemi
author:zcyemi
feat(LinearAlgebra/AffineSpace/Independent): Add affineCombination_eq_lineMap_iff_weight_lineMap --- ```lean theorem AffineIndependent.affineCombination_eq_lineMap_iff_weight_lineMap {p : ι → P} (ha : AffineIndependent k p) {w w₁ w₂ : ι → k} {s : Finset ι} (hw : ∑ i ∈ s, w i = 1) (hw₁ : ∑ i ∈ s, w₁ i = 1) (hw₂ : ∑ i ∈ s, w₂ i = 1) (c : k) : s.affineCombination k p w = AffineMap.lineMap (s.affineCombination k p w₁) (s.affineCombination k p w₂) c ↔ ∀ i ∈ s, w i = AffineMap.lineMap (w₁ i) (w₂ i) c := by ``` This theorem is a parameterized reformulation of `affineCombination_mem_affineSpan_pair`. It is convenient for rewriting when a concrete `lineMap` parameter is given. t-algebra
label:t-algebra$
23/0 Mathlib/LinearAlgebra/AffineSpace/Independent.lean 1 4 ['github-actions', 'jsm28', 'zcyemi'] nobody none
3-25950
3 days ago
3-24253
3 days ago
3-30373
3 days
33863 urkud
author:urkud
feat: generalize some lemmas about LTOs Currently, lemmas about `Filter.map ((↑) : Set.Iio a → X) Filter.atTop` etc assume that the ambient type is densely ordered. However, it suffices to require that `a` is an `Order.IsSuccPrelimit`. Make this generalization and move the lemmas to a new file. Also, use the new lemmas to drop a `[DenselyOrdered _]` assumption in one lemma in measure theory. These more precise statements are also useful when dealing with, e.g., LTOs defined by ordinals. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 226/130 Mathlib.lean,Mathlib/Analysis/SpecialFunctions/Exp.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Arctan.lean,Mathlib/MeasureTheory/Measure/Hausdorff.lean,Mathlib/MeasureTheory/Measure/MeasureSpace.lean,Mathlib/Topology/Order/AtTopBotIxx.lean,Mathlib/Topology/Order/DenselyOrdered.lean 7 1 ['github-actions'] nobody none
3-17889
3 days ago
3-16170
3 days ago
3-15991
3 days

Stale assigned PRs on the review queue

Number Author Title Description Labels +/- Modified files (first 100) 📝 💬 All users who commented or reviewed Assignee(s) Approval(s) Updated Last status change total time in review
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
none
44-31268
1 month ago
47-15803
47 days ago
47-15624
47 days
32124 SnirBroshi
author:SnirBroshi
feat(SimpleGraph/Walks/Operations): expand basic drop/take/reverse API --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics 44/0 Mathlib/Combinatorics/SimpleGraph/Walks/Operations.lean 1 1 ['github-actions'] awainverse
assignee:awainverse
none
44-31258
1 month ago
50-22776
50 days ago
50-22597
50 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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
none
43-31254
1 month ago
47-20681
47 days ago
47-20502
47 days
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta 703/0 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/WildcardLevel.lean,MathlibTest/WildcardLevel.lean 4 25 ['JovanGerb', 'adamtopaz', 'github-actions'] dwrensha
assignee:dwrensha
none
38-31260
1 month ago
40-48971
40 days ago
42-30056
42 days
32455 vihdzp
author:vihdzp
feat: order topologies of successor orders --- Co-authored by @j-loreaux [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology t-order 124/43 Mathlib.lean,Mathlib/Order/Cover.lean,Mathlib/SetTheory/Ordinal/Topology.lean,Mathlib/Topology/Order/SuccPred.lean 4 1 ['github-actions'] pechersky
assignee:pechersky
none
37-31259
1 month ago
41-15158
41 days ago
41-14979
41 days
32552 ksenono
author:ksenono
feat(SetTheory/Cardinal): helpers for Konig's theorem --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-set-theory new-contributor 70/0 Mathlib/SetTheory/Cardinal/Arithmetic.lean,Mathlib/SetTheory/Cardinal/Basic.lean 2 33 ['SnirBroshi', 'b-mehta', 'github-actions', 'ksenono', 'staroperator', 'vihdzp'] b-mehta
assignee:b-mehta
1
32-15388
1 month ago
32-36796
32 days ago
37-79310
37 days
26608 vihdzp
author:vihdzp
feat(SetTheory/Cardinal/Aleph): `o.card ≤ ℵ_ o` and variants --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-set-theory 24/0 Mathlib/SetTheory/Cardinal/Aleph.lean 1 4 ['artie2000', 'github-actions', 'kckennylau', 'leanprover-community-bot-assistant', 'vihdzp'] alreadydone
assignee:alreadydone
2
29-66799
29 days ago
29-74566
29 days ago
59-56107
59 days
32772 tb65536
author:tb65536
feat(Data/Set/Card): criterion for `s.ncard ≤ (f '' s).ncard + 1` This PR gives a criterion `s.ncard ≤ (f '' s).ncard + 1` (note that we always have the inequality `(f '' s).ncard ≤ s.ncard`). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data 31/0 Mathlib/Data/Set/Card.lean 1 1 ['github-actions'] pechersky
assignee:pechersky
none
28-31259
28 days ago
34-14214
34 days ago
34-14035
34 days
32555 ksenono
author:ksenono
feat(Combinatorics/SimpleGraph/Matching): maximum and maximal matchings for Konig's theorem --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics new-contributor 127/1 Mathlib/Combinatorics/SimpleGraph/DegreeSum.lean,Mathlib/Combinatorics/SimpleGraph/Matching.lean 2 8 ['SnirBroshi', 'github-actions', 'ksenono'] awainverse
assignee:awainverse
none
28-19909
28 days ago
28-18982
28 days ago
38-43127
38 days
32570 ksenono
author:ksenono
feat(Combinatorics/SimpleGraph): bipartite subgraphs and vertex-disjoint graphs for Konig's theorem --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics new-contributor 22/0 Mathlib/Combinatorics/SimpleGraph/Bipartite.lean,Mathlib/Combinatorics/SimpleGraph/Subgraph.lean 2 10 ['SnirBroshi', 'github-actions'] kmill
assignee:kmill
1
28-19449
28 days ago
28-18541
28 days ago
38-18442
38 days
32679 YaelDillies
author:YaelDillies
chore(Data/Sym2): improve defeq of `diagSet` #30559 introduced a regression on the defeqs in the `SimpleGraph` API. This PR fixes it. From LeanCamCombi --- I personally think this new `diagSet` definition is unnecessary: `{e | e.IsDiag}` is not much longer to write than `Sym2.diagSet` and more transparent, but whatever. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data 52/41 Mathlib/Combinatorics/SimpleGraph/Basic.lean,Mathlib/Combinatorics/SimpleGraph/DeleteEdges.lean,Mathlib/Combinatorics/SimpleGraph/Operations.lean,Mathlib/Data/Sym/Card.lean,Mathlib/Data/Sym/Sym2.lean 5 9 ['SnirBroshi', 'YaelDillies', 'b-mehta', 'github-actions', 'mathlib4-merge-conflict-bot', 'vihdzp'] pechersky
assignee:pechersky
1
27-42873
27 days ago
27-41047
27 days ago
33-80987
33 days
32532 SnirBroshi
author:SnirBroshi
feat(Combinatorics/SimpleGraph/Connectivity): connected components are maximally connected subsets/subgraphs --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics 32/0 Mathlib/Combinatorics/SimpleGraph/Connectivity/Connected.lean,Mathlib/Combinatorics/SimpleGraph/Connectivity/Subgraph.lean 2 2 ['github-actions', 'mathlib4-merge-conflict-bot'] awainverse
assignee:awainverse
none
26-39490
26 days ago
26-38659
26 days ago
39-5863
39 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`, a direct construction without ε-transitions. - Theorem `accepts_concat : (M1.concat M2).accepts = M1.accepts * M2.accepts`, showing the correctness of the construction. - Theorem `IsRegular.mul`, showing that regular languages are closed under concatenation. --- - [x] depends on: #31038 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-computability new-contributor maintainer-merge 104/7 Mathlib/Computability/NFA.lean 1 63 ['YaelDillies', 'ctchou', 'github-actions', 'lambda-fairy', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'rudynicolop'] YaelDillies
assignee:YaelDillies
2
26-39225
26 days ago
26-38269
26 days ago
45-11894
45 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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-euclidean-geometry 157/0 Mathlib/Geometry/Euclidean/Angle/Oriented/Affine.lean 1 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] JovanGerb
assignee:JovanGerb
none
26-31275
26 days ago
29-41289
29 days ago
29-43242
29 days
32826 felixpernegger
author:felixpernegger
feat(Data/Tuple/Sort): Permutation is monotone iff its the identity Sort of permutation is its inverse + Permutation is monotone iff its the identity t-data new-contributor 19/0 Mathlib/Data/Fin/Tuple/Sort.lean 1 1 ['github-actions'] TwoFX
assignee:TwoFX
none
26-31271
26 days ago
30-75518
30 days ago
33-21577
33 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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) brownian t-measure-probability large-import 111/4 Mathlib/Data/Setoid/Partition.lean,Mathlib/MeasureTheory/Function/SimpleFunc.lean,Mathlib/MeasureTheory/Function/StronglyMeasurable/Basic.lean,Mathlib/MeasureTheory/MeasurableSpace/Basic.lean 4 21 ['CoolRmal', 'EtienneC30', 'github-actions', 'hanwenzhu', 'mathlib4-merge-conflict-bot'] EtienneC30
assignee:EtienneC30
none
25-83406
25 days ago
25-81916
25 days ago
47-53628
47 days
32739 Rida-Hamadani
author:Rida-Hamadani
chore(SimpleGraph): golf and improve style of `Subwalks.lean` maintaining the sub-walks file after the walk split, golfing some proofs --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics 11/18 Mathlib/Combinatorics/SimpleGraph/Walks/Subwalks.lean 1 1 ['github-actions', 'vlad902'] awainverse
assignee:awainverse
1
25-31244
25 days ago
34-179
34 days ago
34-0
34 days
32910 felixpernegger
author:felixpernegger
feat(Data/Nat/Choose): two binomial coefficient sum identities This PR proves two well-known sum identities around binomial coefficients. While there are probably hundreds of such identities, these two seem to be well known enough to be in mathlib (i.e. are mentioned in the Wikipedia [article](https://en.wikipedia.org/wiki/Binomial_coefficient#math_8) about binomial coefficients). new-contributor t-data 31/0 Mathlib/Data/Nat/Choose/Sum.lean,Mathlib/Data/Nat/Choose/Vandermonde.lean 2 1 ['github-actions'] TwoFX
assignee:TwoFX
none
25-31241
25 days ago
30-65060
30 days ago
30-64881
30 days
32989 kim-em
author:kim-em
fix(Tactic/Simps): skip @[defeq] inference for non-exposed definitions This PR makes `@[simps]` check whether the source definition's body is exposed before calling `inferDefEqAttr`. When the body is not exposed, we skip the `@[defeq]` inference to avoid validation errors. Without this fix, using `@[simps]` on a definition that is not `@[expose]`d produces an error like: ``` Theorem Foo_bar has a `rfl`-proof and was thus inferred to be `@[defeq]`, but validating that attribute failed: Not a definitional equality: the left-hand side ... is not definitionally equal to the right-hand side ... Note: This theorem is exported from the current module. This requires that all definitions that need to be unfolded to prove this theorem must be exposed. ``` The fix checks `(← getEnv).setExporting true |>.find? cfg.srcDeclName |>.any (·.hasValue)` to determine if the definition body is visible in the public scope, and only calls `inferDefEqAttr` if it is. 🤖 Prepared with Claude Code t-meta 40/2 Mathlib/Tactic/Simps/Basic.lean,MathlibTest/SimpsModule.lean 2 8 ['JovanGerb', 'github-actions', 'kim-em'] eric-wieser
assignee:eric-wieser
none
25-31240
25 days ago
26-32060
26 days ago
28-81065
28 days
33016 xgenereux
author:xgenereux
feat: RingHom.adjoinAlgebraMap Consider a tower of rings `A / B / C` and `b : B`, then there is a natural map from `A[b]` to `A[algebraMap B C b]` (adjoin `b` viewed as an element of `C`). This PR adds 3 versions, depending on whether we use `Algebra.adjoin` or `IntermediateField.adjoin`: - `Algebra.RingHom.adjoinAlgebraMap : Algebra.adjoin A {b} →+* Algebra.adjoin A {(algebraMap B C) b}` - `IntermediateField.RingHom.adjoinAlgebraMapOfAlgebra : Algebra.adjoin A {b} →+* A⟮((algebraMap B C) b)⟯` - `IntermediateField.RingHom.adjoinAlgebraMap : A⟮b⟯ →+* A⟮((algebraMap B C) b)⟯` Note: We create a new file for `Algebra.RingHom.adjoinAlgebraMap`, which is intended for results about adjoining singletons, because it is convenient to import `Algebra.Adjoin.Polynomial`. Co-authored-by: María Inés de Frutos Fernández <[mariaines.dff@gmail.com](mailto:mariaines.dff@gmail.com)> --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 103/0 Mathlib.lean,Mathlib/FieldTheory/IntermediateField/Adjoin/Algebra.lean,Mathlib/FieldTheory/IntermediateField/Adjoin/Defs.lean,Mathlib/RingTheory/Adjoin/Singleton.lean 4 1 ['github-actions'] bryangingechen
assignee:bryangingechen
none
25-31237
25 days ago
28-37013
28 days ago
28-36834
28 days
30898 vihdzp
author:vihdzp
feat: characterization of `List.splitBy` --- - [x] depends on: #30892 Moved from #16837. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data 110/10 Mathlib/Data/List/Flatten.lean,Mathlib/Data/List/SplitBy.lean 2 6 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'vihdzp'] TwoFX
assignee:TwoFX
none
25-25271
25 days ago
25-22234
25 days ago
34-53081
34 days
26484 peabrainiac
author:peabrainiac
feat(Geometry/Diffeology): basics of diffeological spaces Introduces diffeological spaces, smooth maps between them, the D-topology and the standard diffeology on finite-dimensional normed spaces. --- This PR continues the work from #21969. t-differential-geometry 491/0 Mathlib.lean,Mathlib/Geometry/Diffeology/Basic.lean,docs/references.bib 3 12 ['JovanGerb', 'github-actions', 'grunweg', 'lecopivo', 'mathlib4-merge-conflict-bot', 'peabrainiac'] ocfnash
assignee:ocfnash
none
24-461
24 days ago
25-34232
25 days ago
163-58726
163 days
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-euclidean-geometry 75/0 Mathlib/Geometry/Euclidean/Altitude.lean 1 4 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] JovanGerb
assignee:JovanGerb
none
23-31263
23 days ago
26-56740
26 days ago
26-56561
26 days
33031 chiyunhsu
author:chiyunhsu
feat(Combinatorics/Enumerative/Partition): add combinatorial proof of Euler's partition theorem The new file EulerComb.lean contains the combinatorial proof of Euler's partition theorem. The analytic proof of the theorem and its generalization of Glaisher's Theorem has already been formalized in [Glaisher.lean](https://github.com/leanprover-community/mathlib4/blob/master/Mathlib/Combinatorics/Enumerative/Partition/Glaisher.lean). The generalization of the combinatorial proof from this file to Glaisher's Theorem is within reach. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics new-contributor 531/0 Mathlib.lean,Mathlib/Combinatorics/Enumerative/Partition/EulerComb.lean 2 5 ['chiyunhsu', 'github-actions', 'tb65536', 'vihdzp'] b-mehta
assignee:b-mehta
none
23-31260
23 days ago
28-3016
28 days ago
28-2837
28 days
33082 AntoineChambert-Loir
author:AntoineChambert-Loir
feat(GroupTheory/SpecificGroups/Alternating/Simple): the alternating group on at least 5 letters is simple. This is the conclusion of the story of the proof of simplicity of the alternating group using the Iwasawa criterion. * `Equiv.Perm.iwasawaStructure_two`: the natural `IwasawaStructure` of `Equiv.Perm α` acting on `Nat.Combination α 2` Its commutative subgroups consist of the permutations with support in a given element of `Nat.Combination α 2`. They are cyclic of order 2. * `alternatingGroup_of_le_of_normal`: If `α` has at least 5 elements, then a nontrivial normal subgroup of `Equiv.Perm α` contains the alternating group. * `alternatingGroup.iwasawaStructure_three`: the natural `IwasawaStructure` of `alternatingGroup α` acting on `Nat.Combination α 3` Its commutative subgroups consist of the permutations with support in a given element of `Nat.Combination α 2`. They are cyclic of order 3. * `alternatingGroup.iwasawaStructure_three`: the natural `IwasawaStructure` of `alternatingGroup α` acting on `Nat.Combination α 4` Its commutative subgroups consist of the permutations of cycleType (2, 2) with support in a given element of `Nat.Combination α 2`. They have order 4 and exponent 2 (`IsKleinFour`). * `alternatingGroup.normal_subgroup_eq_bot_or_eq_top`: If `α` has at least 5 elements, then a nontrivial normal subgroup of `alternatingGroup` is `⊤`. * `alternatingGroup.isSimpleGroup`: If `α` has at least 5 elements, then `alternatingGroup α` is a simple group. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-group-theory large-import 821/13 Mathlib.lean,Mathlib/GroupTheory/GroupAction/SubMulAction/Combination.lean,Mathlib/GroupTheory/Perm/Cycle/Type.lean,Mathlib/GroupTheory/Perm/Support.lean,Mathlib/GroupTheory/SpecificGroups/Alternating.lean,Mathlib/GroupTheory/SpecificGroups/Alternating/Simple.lean,Mathlib/GroupTheory/SpecificGroups/KleinFour.lean 7 1 ['github-actions'] mattrobball
assignee:mattrobball
none
23-31255
23 days ago
26-59667
26 days ago
26-59488
26 days
33109 felixpernegger
author:felixpernegger
feat(Data/Nat/Choose): Binomial inversion This PR adds binomial inversion (also called binomial transform), which is a useful method for proving binomial identities. It is tricky to find direct references to binomial inversion, but for example [this](https://en.wikipedia.org/wiki/Binomial_transform#Binomial_convolution) Wikipedia article mentions it ("The formula"). The first theorem ```alternating_sum_choose_mul_of_alternating_sum_choose_mul``` could be refined (we only need the hypothesis ```h``` up to some point), but this seems to needlessly complicate it. new-contributor 107/0 Mathlib.lean,Mathlib/Data/Nat/Choose/Inversion.lean 2 4 ['felixpernegger', 'github-actions', 'wwylele'] dagurtomas
assignee:dagurtomas
none
23-31250
23 days ago
25-62271
25 days ago
26-4033
26 days
33126 CoolRmal
author:CoolRmal
feat: function composition preserves boundedness This PR adds the following theorem: if the range of a function `g` is bounded above, then `g ∘ f` is bounded above for all functions `f`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order 12/0 Mathlib/Order/Bounds/Basic.lean 1 1 ['github-actions'] bryangingechen
assignee:bryangingechen
none
22-31251
22 days ago
25-71899
25 days ago
25-71720
25 days
32160 SnirBroshi
author:SnirBroshi
feat(Combinatorics/SimpleGraph/Walks): helper theorems about `darts` and `support` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics 33/1 Mathlib/Combinatorics/SimpleGraph/Walks/Basic.lean,Mathlib/Combinatorics/SimpleGraph/Walks/Traversal.lean 2 1 ['github-actions'] kmill
assignee:kmill
none
21-46913
21 days ago
21-46053
21 days ago
49-22904
49 days
33147 SnirBroshi
author:SnirBroshi
feat(Combinatorics/SimpleGraph/Coloring): add a few missing instances (`IsEmpty`/`Nontrivial`/`Infinite`) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics 22/0 Mathlib/Combinatorics/SimpleGraph/Coloring.lean,Mathlib/Combinatorics/SimpleGraph/Maps.lean 2 1 ['github-actions'] b-mehta
assignee:b-mehta
none
21-31265
21 days ago
25-23535
25 days ago
25-23356
25 days
31092 FlAmmmmING
author:FlAmmmmING
feat(Algebra/Group/ForwardDiff.lean): Add theorem `sum_shift_eq_fwdDiff_iter`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra new-contributor
label:t-algebra$
17/1 Mathlib/Algebra/Group/ForwardDiff.lean 1 18 ['BeibeiX0', 'FlAmmmmING', 'Ruben-VandeVelde', 'dagurtomas', 'github-actions', 'mathlib4-merge-conflict-bot'] dagurtomas
assignee:dagurtomas
none
21-6633
21 days ago
21-5472
21 days ago
46-81323
46 days
33121 SnirBroshi
author:SnirBroshi
feat(Combinatorics/SimpleGraph/Hasse): paths in a graph are isomorphic to path graphs --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics large-import 38/1 Mathlib/Combinatorics/SimpleGraph/Hasse.lean 1 1 ['github-actions'] b-mehta
assignee:b-mehta
none
20-79234
20 days ago
20-78269
20 days ago
25-84611
25 days
33211 Komyyy
author:Komyyy
doc(Order/Filter/*): outdated documents `f ×ˢ g` is not an notation of `Filter.prod` anymore, but [a notation class](https://leanprover-community.github.io/mathlib4_docs/Mathlib/Order/Filter/Defs.html#Filter.instSProd). Also, some definitions were moved to `Mathlib.Order.Filter.Defs`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) documentation t-order 6/10 Mathlib/Order/Filter/Curry.lean,Mathlib/Order/Filter/Pi.lean,Mathlib/Order/Filter/Prod.lean 3 6 ['Komyyy', 'github-actions', 'plp127'] bryangingechen
assignee:bryangingechen
none
20-31254
20 days ago
21-26898
21 days ago
23-30281
23 days
33248 vihdzp
author:vihdzp
refactor(MeasureTheory/Measure/Stieltjes): simpler definition of `botSet` --- Arguably we could get rid of `botSet` altogether, but in either case this is still an improvement. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-measure-probability 13/19 Mathlib/MeasureTheory/Measure/Stieltjes.lean 1 1 ['github-actions'] EtienneC30
assignee:EtienneC30
none
19-31259
19 days ago
21-65986
21 days ago
21-65916
21 days
32987 kim-em
author:kim-em
feat: pipeline downloads and decompression in `cache get` This PR modifies `lake exe cache get` to decompress files as they download, rather than waiting for all downloads to complete first. Previously the cache system had two sequential phases: download all files using `curl --parallel`, then decompress all files using a single `leantar` call. Now a background task spawns sequential batched `leantar` calls to decompress files as downloads complete, pipelining network I/O and disk I/O. 🤖 Prepared with Claude Code 194/30 Cache/Requests.lean 1 1 ['github-actions'] dagurtomas
assignee:dagurtomas
none
18-31229
18 days ago
28-32214
28 days ago
29-29019
29 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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import 227/2 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
none
17-33855
17 days ago
17-31508
17 days ago
64-13257
64 days
33280 michelsol
author:michelsol
feat(MeasureTheory/Integral/IntervalIntegral): add variant `integral_deriv_eq_sub_uIoo` of 2nd theorem of calculus. Add a continuous on uIcc, differentiable on uIoo, deriv version of the 2nd fundamental theorem of calculus. This corresponds to what is written [here](https://en.wikipedia.org/wiki/Fundamental_theorem_of_calculus#Second_part). For example it makes it easier to compute the integral : ```lean4 ∫ x : ℝ in 0..1, (√(1 - x ^ 2))⁻¹ = ∫ x : ℝ in 0..1, deriv arcsin x = arcsin 1 - arcsin 0 ``` It is not possible to use [`interval_deriv_eq_sub`](https://leanprover-community.github.io/mathlib4_docs/Mathlib/MeasureTheory/Integral/IntervalIntegral/FundThmCalculus.html#intervalIntegral.integral_deriv_eq_sub) which requires differentiability on all of [0,1], as `arcsin` isn't differentiable at 1. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-measure-probability new-contributor 14/0 Mathlib/MeasureTheory/Integral/IntervalIntegral/FundThmCalculus.lean 1 1 ['github-actions'] EtienneC30
assignee:EtienneC30
none
17-31242
17 days ago
20-55887
20 days ago
20-55708
20 days
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 45 ['BoltonBailey', 'IlPreteRosso', 'TwoFX', 'github-actions', 'kckennylau', 'mathlib4-merge-conflict-bot', 'rudynicolop'] TwoFX
assignee:TwoFX
none
17-20160
17 days ago
26-38101
26 days ago
90-59512
90 days
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`. t-combinatorics new-contributor 76/0 Mathlib.lean,Mathlib/Combinatorics/Enumerative/RecLatticePath.lean 2 3 ['github-actions', 'mathlib4-merge-conflict-bot'] awainverse
assignee:awainverse
none
16-83519
16 days ago
16-82696
16 days ago
36-28736
36 days
33064 DavidLedvinka
author:DavidLedvinka
feat(Probability): Add `condLExp`, conditional expectation with the Lebesgue integral Add definition of `condLExp`, conditional expectation using the Lebesgue integral. Also add basic API. t-measure-probability 275/0 Mathlib.lean,Mathlib/MeasureTheory/Function/ConditionalLExpectation.lean,Mathlib/MeasureTheory/Integral/Lebesgue/Add.lean,Mathlib/MeasureTheory/MeasurableSpace/CountablyGenerated.lean,Mathlib/MeasureTheory/MeasurableSpace/Defs.lean,Mathlib/MeasureTheory/Measure/AEMeasurable.lean 6 3 ['DavidLedvinka', 'github-actions', 'leanprover-radar'] EtienneC30
assignee:EtienneC30
none
16-36441
16 days ago
16-35563
16 days ago
26-38803
26 days
33143 wwylele
author:wwylele
feat(PowerSeries): pentagonal number theorem The proof is split in two files: `Mathlib/Topology/Algebra/InfiniteSum/Pentagonal.lean` for the algebraic part, and `Mathlib/RingTheory/PowerSeries/Pentagonal.lean` for the summability part. In the near future, I also plan to prove the real/complex version that branches off from the algebraic part. --- - [ ] depends on: #30436 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 324/1 Mathlib.lean,Mathlib/RingTheory/PowerSeries/Pentagonal.lean,Mathlib/Topology/Algebra/InfiniteSum/Pentagonal.lean,docs/1000.yaml 4 12 ['copilot-pull-request-reviewer', 'github-actions', 'mathlib4-dependent-issues-bot', 'vihdzp'] kex-y
assignee:kex-y
none
16-31260
16 days ago
18-69043
18 days ago
19-38681
19 days
33297 tb65536
author:tb65536
feat(Algebra/Polynomial/Roots): add `card_rootSet_le` This PR adds a lemma stating that `Set.ncard (p.rootSet B) ≤ p.natDegree` (we already have similar lemmas for `Polynomial.roots`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra large-import
label:t-algebra$
7/0 Mathlib/Algebra/Polynomial/Roots.lean 1 1 ['github-actions'] dagurtomas
assignee:dagurtomas
none
16-31259
16 days ago
20-27259
20 days ago
20-27080
20 days

PRs with just failing CI, but only often-spurious jobs

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
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 t-algebra merge-conflict slow-typeclass-synthesis awaiting-zulip t-analysis
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
134-35234
4 months ago
142-72788
142 days ago
0-16864
4 hours
29514 grunweg
author:grunweg
feat(CI): use more strict mode --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP CI 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
56-64957
1 month ago
unknown
unknown
33766 alreadydone
author:alreadydone
feat(Analysis, Topology): more examples of covering maps involving the complex plane --- - [ ] depends on: #33726 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-topology t-analysis blocked-by-other-PR large-import 311/11 Mathlib/Algebra/Polynomial/Eval/Defs.lean,Mathlib/Algebra/Polynomial/Roots.lean,Mathlib/Analysis/Complex/CoveringMap.lean,Mathlib/Analysis/Complex/OpenMapping.lean,Mathlib/Analysis/SpecialFunctions/Complex/Circle.lean,Mathlib/Data/Nat/Init.lean,Mathlib/FieldTheory/IsAlgClosed/Basic.lean,Mathlib/RingTheory/RootsOfUnity/Basic.lean,Mathlib/Topology/Algebra/GroupWithZero.lean,Mathlib/Topology/Algebra/Polynomial.lean,Mathlib/Topology/Covering/Basic.lean 11 4 ['alreadydone', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
1-36765
1 day ago
unknown
unknown
32777 madvorak
author:madvorak
doc: Contributing moved to Contributing --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 54/56 .github/CONTRIBUTING.md,README.md 2 2 ['github-actions'] Vierkantor
assignee:Vierkantor
1-31239
1 day ago
34-4535
34 days ago
34-4356
34 days
33765 JovanGerb
author:JovanGerb
feat(Order/CompleteLattice/Defs): `to_dual` for `CompleteSemilattice`s This PR uses `to_dual` for `CompleteSemilatticeSup` and `CompleteSemilatticeInf`. These will need to be refactored/deprecated in the future, but I think it makes sense to make the code smaller (using `to_dual`) before such a refactor. --- - [ ] depends on: #33760 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR large-import t-order 157/360 Mathlib/Order/Bounds/Basic.lean,Mathlib/Order/Bounds/Defs.lean,Mathlib/Order/CompleteLattice/Defs.lean,Mathlib/Order/Interval/Set/Defs.lean,Mathlib/Tactic/Translate/ToDual.lean 5 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'vihdzp'] nobody
1-3549
1 day ago
unknown
unknown
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? [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) delegated t-meta 55/14 Mathlib/Tactic/Abel.lean,Mathlib/Tactic/FieldSimp.lean,Mathlib/Tactic/Ring/RingNF.lean,Mathlib/Util/AtomM/Recurse.lean,MathlibTest/FieldSimp.lean 5 29 ['FLDutchmann', 'JovanGerb', 'Vierkantor', 'github-actions', 'grunweg', 'leanprover-radar', 'mathlib-bors'] alexjbest
assignee:alexjbest
0-78358
21 hours ago
0-78358
21 hours ago
26-19830
26 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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author new-contributor t-order 255/0 Mathlib.lean,Mathlib/Algebra/BigOperators/Group/Finset/Gaps.lean,Mathlib/Order/Interval/Finset/Gaps.lean 3 6 ['github-actions', 'sgouezel', 'zhuyizheng'] sgouezel
assignee:sgouezel
0-72016
20 hours ago
0-82276
22 hours ago
48-35273
48 days

PRs addressing technical debt

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
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-linter tech debt 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
533-5307
1 year ago
unknown
unknown
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`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-computability tech debt 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
514-48092
1 year ago
unknown
unknown
15448 urkud
author:urkud
chore(*): deprecate `Option.elim'` Use `Option.elim` instead. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author tech debt 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
513-58057
1 year ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-linter awaiting-author tech debt 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
350-47266
11 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict tech debt t-topology RFC 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
289-19886
9 months ago
unknown
unknown
24100 eric-wieser
author:eric-wieser
feat: restore some explicit binders from Lean 3 Part of #24099 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author tech debt 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
234-70460
7 months 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. merge-conflict awaiting-author tech debt t-analysis 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 10 ['ADedecker', 'b-mehta', 'github-actions', 'j-loreaux', 'mathlib4-merge-conflict-bot', 'mcdoll', 'plp127'] nobody
61-68331
2 months ago
64-55703
64 days ago
2-74132
2 days
33138 gasparattila
author:gasparattila
chore(MeasureTheory/Measure/Stieltjes): remove `backward.privateInPublic` In #32482, some definitions in this file were rewritten using private declarations. However, this made `StieltjesFunction.length` unusable, since its API uses private declarations even in statements. This PR fixes this by problem by specializing `length_eq` to `NoMinOrder` and adding a new lemma for the `OrderBot` case. The other lemmas involving the private declarations are made private, except for `length_subadditive_Icc_Ioo`, which is reverted to the previous statement. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-measure-probability tech debt awaiting-author 35/30 Mathlib/MeasureTheory/Measure/Stieltjes.lean 1 6 ['github-actions', 'grunweg', 'sgouezel', 'vihdzp'] sgouezel
assignee:sgouezel
20-42330
20 days ago
20-42330
20 days ago
5-472
5 days
33921 SnirBroshi
author:SnirBroshi
chore(Data/Nat/Factorial): replace `n !` with `(n)!` everywhere Fixes ``Todo: replace occurrences of `n !` with `(n)!` in Mathlib.`` from `Data/Nat/Factorial/Basic.lean`. Only literals are allowed to use factorial unparenthesized, e.g. `5!`. --- The TODO was introduced in #18085, with an accompanying [Zulip discussion](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/precedence.20of.20Nat.2Efactorial) that decided on this. The factorial notation is used in Mathlib on the following kinds of expressions: - `Nat` numerals, e.g. `5`, there are 20 such cases - Identifiers, e.g. `n` or `n.succ` or `l.length` or `p.natDegree`, there are 433 such cases - Structure projection, e.g. `n.1`, there are 20 such cases - Parenthesized expressions, e.g. `(n + k)`, there are 293 such cases - Type ascriptions, e.g. `(n : ℕ)` (these don't count as parenthesized in `Lean.Syntax`), there are [3](https://github.com/leanprover-community/mathlib4/blob/b2f24e70b375e42e5a60251a2f43baa20ca668f1/MathlibTest/norm_num_ext.lean#L625) [such](https://github.com/leanprover-community/mathlib4/blob/b2f24e70b375e42e5a60251a2f43baa20ca668f1/Mathlib/MeasureTheory/Measure/Lebesgue/VolumeOfBalls.lean#L378) [cases](https://github.com/leanprover-community/mathlib4/blob/b2f24e70b375e42e5a60251a2f43baa20ca668f1/Mathlib/MeasureTheory/Measure/Lebesgue/VolumeOfBalls.lean#L384) This PR normalizes everything to use `(...)!` notation, except for numerals which don't require parentheses. Note that structure projections also don't require parentheses but it looks confusing (see [this](https://github.com/leanprover-community/mathlib4/blob/4baa44807be87d9aba67c680ae68c2ba4a7fc29b/Mathlib/Data/Nat/Factorial/NatCast.lean#L106) and [this](https://github.com/leanprover-community/mathlib4/blob/4baa44807be87d9aba67c680ae68c2ba4a7fc29b/Mathlib/NumberTheory/Bernoulli.lean#L150)), so parentheses were added. I used metaprogramming + Python to create this PR; these are the non-formulaic changes: - Deleted the TODO in `Data/Nat/Factorial/Basic.lean` - Fixed 3 comments in `Data/Nat/Factorial/Basic.lean` that used ` !` - The replacement caused these lines to go over the length limit, so I fixed them manually: - `Archive/Imo/Imo2019Q4.lean:84` - `Mathlib/Data/Nat/Choose/Basic.lean:289` - `Mathlib/RingTheory/DividedPowers/RatAlgebra.lean:134` - `Mathlib/RingTheory/Polynomial/ShiftedLegendre.lean:71` In a future PR I'll add a linter that requires parentheses inside factorials for non-numerals, then the whitespace linter will lint against spaces between `)` and `!`. (though the pretty printer's parenthesizer still prefers adding spaces instead of parentheses, not sure how to fix it) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) tech debt t-data 402/401 Archive/Imo/Imo1987Q1.lean,Archive/Imo/Imo2001Q4.lean,Archive/Imo/Imo2019Q4.lean,Mathlib/Algebra/BigOperators/Intervals.lean,Mathlib/Algebra/Group/ForwardDiff.lean,Mathlib/Algebra/Polynomial/Derivative.lean,Mathlib/Algebra/Polynomial/FieldDivision.lean,Mathlib/Algebra/Polynomial/HasseDeriv.lean,Mathlib/Algebra/Polynomial/SumIteratedDerivative.lean,Mathlib/Analysis/Analytic/Binomial.lean,Mathlib/Analysis/Calculus/ContDiff/Bounds.lean,Mathlib/Analysis/Calculus/Deriv/ZPow.lean,Mathlib/Analysis/Calculus/FDeriv/Analytic.lean,Mathlib/Analysis/Calculus/IteratedDeriv/WithinZpow.lean,Mathlib/Analysis/Calculus/Taylor.lean,Mathlib/Analysis/Complex/Exponential.lean,Mathlib/Analysis/Complex/TaylorSeries.lean,Mathlib/Analysis/Distribution/SchwartzSpace.lean,Mathlib/Analysis/Distribution/TemperateGrowth.lean,Mathlib/Analysis/Normed/Algebra/Exponential.lean,Mathlib/Analysis/ODE/PicardLindelof.lean,Mathlib/Analysis/Real/Pi/Irrational.lean,Mathlib/Analysis/Real/Pi/Wallis.lean,Mathlib/Analysis/SpecialFunctions/Exp.lean,Mathlib/Analysis/SpecialFunctions/Gamma/Basic.lean,Mathlib/Analysis/SpecialFunctions/Gamma/Beta.lean,Mathlib/Analysis/SpecialFunctions/Gamma/BohrMollerup.lean,Mathlib/Analysis/SpecialFunctions/OrdinaryHypergeometric.lean,Mathlib/Analysis/SpecialFunctions/Stirling.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Cotangent.lean,Mathlib/Analysis/SpecificLimits/Basic.lean,Mathlib/Analysis/SpecificLimits/Normed.lean,Mathlib/Combinatorics/Enumerative/Bell.lean,Mathlib/Data/Fintype/Perm.lean,Mathlib/Data/List/Permutation.lean,Mathlib/Data/Nat/Choose/Basic.lean,Mathlib/Data/Nat/Choose/Bounds.lean,Mathlib/Data/Nat/Choose/Cast.lean,Mathlib/Data/Nat/Choose/Factorization.lean,Mathlib/Data/Nat/Choose/Multinomial.lean,Mathlib/Data/Nat/Factorial/Basic.lean,Mathlib/Data/Nat/Factorial/BigOperators.lean,Mathlib/Data/Nat/Factorial/DoubleFactorial.lean,Mathlib/Data/Nat/Factorial/NatCast.lean,Mathlib/Data/Nat/Factorial/SuperFactorial.lean,Mathlib/Data/Nat/Multiplicity.lean,Mathlib/Data/Nat/Prime/Factorial.lean,Mathlib/Data/Nat/Prime/Infinite.lean,Mathlib/Data/ZMod/Factorial.lean,Mathlib/GroupTheory/IndexNormal.lean,Mathlib/GroupTheory/Perm/Centralizer.lean,Mathlib/NumberTheory/Bernoulli.lean,Mathlib/NumberTheory/BernoulliPolynomials.lean,Mathlib/NumberTheory/Harmonic/GammaDeriv.lean,Mathlib/NumberTheory/ModularForms/EisensteinSeries/QExpansion.lean,Mathlib/NumberTheory/Padics/PadicVal/Basic.lean,Mathlib/NumberTheory/PrimesCongruentOne.lean,Mathlib/NumberTheory/Transcendental/Lindemann/AnalyticalPart.lean,Mathlib/NumberTheory/Transcendental/Liouville/LiouvilleNumber.lean,Mathlib/NumberTheory/ZetaValues.lean,Mathlib/Probability/Distributions/Poisson.lean,Mathlib/Probability/Moments/MGFAnalytic.lean,Mathlib/RingTheory/DividedPowers/Basic.lean,Mathlib/RingTheory/DividedPowers/Padic.lean,Mathlib/RingTheory/DividedPowers/RatAlgebra.lean,Mathlib/RingTheory/Nilpotent/Exp.lean,Mathlib/RingTheory/Polynomial/HilbertPoly.lean,Mathlib/RingTheory/Polynomial/Pochhammer.lean,Mathlib/RingTheory/Polynomial/ShiftedLegendre.lean,Mathlib/RingTheory/PowerSeries/WellKnown.lean,Mathlib/Tactic/NormNum/NatFactorial.lean,Mathlib/Topology/Algebra/Order/Floor.lean,MathlibTest/GCongr/inequalities.lean,MathlibTest/Simproc/Divisors.lean,MathlibTest/factorial.lean,MathlibTest/norm_num_ext.lean,MathlibTest/positivity.lean 77 1 ['github-actions'] nobody
0-73378
20 hours ago
1-552
1 day ago
1-373
1 day
33896 loefflerd
author:loefflerd
refactor(Geometry/Manifold): split long file ChartedSpace.lean Split the > 1500 line file `Mathlib.Geometry.Manifold.ChartedSpace` into 3 shorter files. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-differential-geometry tech debt ready-to-merge 935/868 Mathlib.lean,Mathlib/Geometry/Manifold/ChartedSpace.lean,Mathlib/Geometry/Manifold/ConformalGroupoid.lean,Mathlib/Geometry/Manifold/HasGroupoid.lean,Mathlib/Geometry/Manifold/IsManifold/Basic.lean,Mathlib/Geometry/Manifold/LocalInvariantProperties.lean,Mathlib/Geometry/Manifold/StructureGroupoid.lean 7 2 ['github-actions', 'jcommelin'] grunweg
assignee:grunweg
0-1635
27 minutes ago
0-1635
24 minutes ago
2-30387
2 days

PRs blocked on a zulip discussion

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
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 merge-conflict t-linter blocked-by-other-PR awaiting-zulip 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
438-57594
1 year ago
unknown
unknown
17623 astrainfinita
author:astrainfinita
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra awaiting-zulip t-order
label:t-algebra$
146/44 Mathlib/Algebra/Order/GroupWithZero/Canonical.lean,Mathlib/Algebra/Order/GroupWithZero/Unbundled.lean 2 11 ['YaelDillies', 'astrainfinita', 'github-actions', 'j-loreaux'] nobody
420-77125
1 year 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) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) This is started from the mathport output on https://github.com/leanprover-community/mathlib/pull/19244 merge-conflict t-analysis awaiting-zulip 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
265-32502
8 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR new-contributor t-computability merge-conflict awaiting-zulip 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
254-40402
8 months ago
unknown
unknown
23929 meithecatte
author:meithecatte
feat(Computability/NFA): improve bound on pumping lemma --- - [x] depends on: #25321 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-computability awaiting-zulip 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
221-50004
7 months ago
221-50005
221 days ago
0-37135
10 hours
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra awaiting-zulip
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
194-20751
6 months ago
unknown
unknown
25218 kckennylau
author:kckennylau
feat(AlgebraicGeometry): Tate normal form of elliptic curves --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebraic-geometry awaiting-zulip new-contributor 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
194-19589
6 months ago
unknown
unknown
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 t-algebra merge-conflict slow-typeclass-synthesis awaiting-zulip t-analysis
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
134-35234
4 months ago
142-72788
142 days ago
0-16864
4 hours
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! [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict file-removed awaiting-zulip 0/564 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/LinearCombination'.lean,Mathlib/Tactic/Linter/UnusedTactic.lean,MathlibTest/linear_combination'.lean 5 4 ['euprunin', 'github-actions', 'grunweg', 'mathlib4-merge-conflict-bot'] nobody
91-12444
2 months ago
unknown
unknown
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) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-linter awaiting-zulip 1/1 Mathlib/Tactic/Linter/Style.lean 1 1 ['github-actions'] nobody
81-46568
2 months ago
unknown
unknown
22361 rudynicolop
author:rudynicolop
feat(Computability/NFA): nfa closure properties Add the closure properties union, intersection and reversal for NFA. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-computability merge-conflict awaiting-author awaiting-zulip 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
72-22134
2 months ago
unknown
unknown
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` [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory large-import new-contributor merge-conflict awaiting-zulip t-meta 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
63-23318
2 months ago
103-1984
103 days ago
0-29227
8 hours
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-computability merge-conflict awaiting-author awaiting-zulip 307/5 Mathlib/Computability/NFA.lean 1 27 ['TpmKranz', 'YaelDillies', 'dupuisf', 'github-actions', 'leanprover-community-bot-assistant', 'meithecatte', 'rudynicolop'] nobody
58-40450
1 month ago
unknown
unknown
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] [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-computability merge-conflict awaiting-author awaiting-zulip 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
57-56691
1 month ago
unknown
unknown
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-computability merge-conflict awaiting-author awaiting-zulip 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
57-55781
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-computability awaiting-zulip new-contributor 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
57-7459
1 month ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) please-adopt merge-conflict t-topology awaiting-zulip 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
56-65725
1 month ago
unknown
unknown
28141 YaelDillies
author:YaelDillies
chore: deprecate `BialgHom.coe_toLinearMap` `BialgHom.toLinearMap` is a fake projection. From Toric --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-ring-theory awaiting-zulip toric 5/11 Mathlib/RingTheory/Bialgebra/Hom.lean 1 16 ['YaelDillies', 'erdOne', 'eric-wieser', 'github-actions'] alreadydone
assignee:alreadydone
53-75570
1 month ago
53-75570
53 days ago
100-70827
100 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`. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data awaiting-author awaiting-zulip 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
49-6247
1 month ago
49-6247
49 days ago
35-75966
35 days
30668 astrainfinita
author:astrainfinita
feat: `QuotType` This typeclass is primarily for use by type synonyms of `Quot` and `Quotient`. Using `QuotType` 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. [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 RFC t-data awaiting-zulip 629/0 Mathlib.lean,Mathlib/Data/QuotType.lean,MathlibTest/QuotType.lean 3 20 ['YaelDillies', 'astrainfinita', 'github-actions', 'mathlib4-merge-conflict-bot', 'plp127', 'vihdzp'] nobody
35-47571
1 month ago
unknown
unknown
32608 PrParadoxy
author:PrParadoxy
feat(LinearAlgebra/PiTensorProduct): API for PiTensorProducts indexed by sets This PR addresses a TODO item in LinearAlgebra/PiTensorProduct.lean: * API for the various ways ι can be split into subsets; connect this with the binary tensor product -- specifically by describing tensors of type ⨂ (i : S), M i, for S : Set ι. Our primary motivation is to formalise the notion of "restricted tensor products". This will be the content of a follow-up PR. Beyond that, the Set API is natural in contexts where the index type has an independent interpretation. An example is quantum physics, where ι ranges over distinguishable degrees of freedom, and where its is common practice to annotate objects by the set of indices they are defined on. --- Stub file with preliminary definition of the restricted tensor product as a direct limit of tensors indexed by finite subsets of an index type: https://github.com/PrParadoxy/mathlib4/blob/restricted-stub/Mathlib/LinearAlgebra/PiTensorProduct/Restricted.lean --- - [x] depends on: #32598 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor awaiting-zulip 300/2 Mathlib.lean,Mathlib/LinearAlgebra/PiTensorProduct.lean,Mathlib/LinearAlgebra/PiTensorProduct/Set.lean 3 28 ['PrParadoxy', 'dagurtomas', 'eric-wieser', 'github-actions', 'goliath-klein', 'leanprover-radar', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] dagurtomas
assignee:dagurtomas
11-59341
11 days ago
23-59044
23 days ago
10-63624
10 days
32742 LTolDe
author:LTolDe
feat(MeasureTheory/Constructions/Polish/Basic): add class SuslinSpace add new class `SuslinSpace` for a topological space that is an analytic set in itself This will be useful to prove the **Effros Theorem**, see [zulip thread](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Effros.20Theorem/with/558712441). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor awaiting-zulip 4/0 Mathlib/MeasureTheory/Constructions/Polish/Basic.lean 1 9 ['ADedecker', 'LTolDe', 'dupuisf', 'github-actions', 'jcommelin'] PatrickMassot
assignee:PatrickMassot
8-65926
8 days ago
8-66079
8 days ago
11-6345
11 days
33368 urkud
author:urkud
feat: define `Complex.UnitDisc.shift` Also review the existing API UPD: I'm going to define a `PSL(2, Real)` action instead. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis awaiting-zulip merge-conflict 273/39 Mathlib.lean,Mathlib/Analysis/Complex/UnitDisc/Basic.lean,Mathlib/Analysis/Complex/UnitDisc/Shift.lean 3 7 ['github-actions', 'j-loreaux', 'mathlib4-merge-conflict-bot', 'sgouezel', 'urkud'] j-loreaux
assignee:j-loreaux
8-15884
8 days ago
8-62617
8 days ago
6-73017
6 days
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'` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-zulip t-logic 78/72 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,Mathlib/RingTheory/Congruence/Hom.lean 8 9 ['SnirBroshi', 'github-actions', 'mathlib4-merge-conflict-bot', 'thorimur', 'vihdzp'] thorimur
assignee:thorimur
4-25105
4 days ago
84-31823
84 days ago
8-45935
8 days

PRs with just a merge conflict

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
24823 eric-wieser
author:eric-wieser
refactor: add `hom` lemmas for the `MonoidalCategory` structure on `ModuleCat` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra
label:t-algebra$
148/164 Mathlib/Algebra/Category/FGModuleCat/Basic.lean,Mathlib/Algebra/Category/ModuleCat/Adjunctions.lean,Mathlib/Algebra/Category/ModuleCat/Monoidal/Basic.lean,Mathlib/Algebra/Category/ModuleCat/Monoidal/Closed.lean,Mathlib/Algebra/Category/ModuleCat/Monoidal/Symmetric.lean,Mathlib/Algebra/Category/ModuleCat/Presheaf/Free.lean,Mathlib/Algebra/Category/ModuleCat/Presheaf/Generator.lean,Mathlib/Algebra/Category/ModuleCat/Presheaf/Monoidal.lean,Mathlib/CategoryTheory/Monoidal/Internal/Module.lean,Mathlib/RepresentationTheory/Coinvariants.lean,Mathlib/RepresentationTheory/Rep.lean 11 21 ['101damnations', 'YaelDillies', 'eric-wieser', 'github-actions', 'joelriou', 'kbuzzard', 'leanprover-community-bot-assistant'] 101damnations
assignee:101damnations
194-19838
6 months ago
194-19838
194 days ago
25-46309
25 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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-topology 18/0 Mathlib/Topology/StoneCech.lean 1 2 ['github-actions', 'leanprover-community-bot-assistant'] nobody
191-658
6 months ago
191-658
191 days ago
20-8050
20 days
9820 jjaassoonn
author:jjaassoonn
feat(RingTheory/GradedAlgebra/HomogeneousIdeal): generalize to homogeneous submodule The definitions, constructions and theorems in `HomogeneousIdeal.lean` are generalized to a homogeneous submodules. So say $R$ is a ring and $M \cong \bigoplus_{i} M_i$ is an $R$-module. Then a homogeneous $R$-submodule of $M$ is an $R$-submodule $N$ such that for all $i$ and $n \in N$, $n_i \in N$. Note that this notion doesn't actually require $R$ to be graded and $M$ is a graded module. But for more interesting lemmas, we do need that $M$ is graded $R$-module. We bake the fact $R$ is graded into the definition of homogeneous submodule, otherwise, `CompleteLattice HomogeneousSubmodule` cannot find the order of synthesis (the proof depends on that $R$ is graded) All definitions/constructions/theorems have a copy for ideals as well, this is to make sure dot notation still works. The motivation of this generalization is graded quotient module --- - [ ] depends on:#18728 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-ring-theory 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
162-86242
5 months ago
unknown
unknown
26200 adomani
author:adomani
fix: add label when landrun fails Adds the `permission-denied` label on PRs that get blocked by landrun. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict CI 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
162-35273
5 months ago
162-35273
162 days ago
46-51722
46 days
27451 kckennylau
author:kckennylau
feat(RingTheory/Valuation): define ball, closed ball, and sphere *From the 2025 Local Class Field Theory Workshop.* --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-ring-theory 27/0 Mathlib/RingTheory/Valuation/Basic.lean 1 13 ['JovanGerb', 'github-actions', 'kckennylau', 'mathlib4-merge-conflict-bot', 'pechersky', 'wwylele'] nobody
156-67776
5 months ago
156-67777
156 days ago
17-51735
17 days
27987 kckennylau
author:kckennylau
feat(RingTheory/Valuation): define ball, closed ball, and sphere --- The pullback PR of #26827 and #27451. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-ring-theory large-import 73/0 Mathlib/RingTheory/Valuation/Basic.lean 1 4 ['JovanGerb', 'github-actions', 'kckennylau', 'mathlib4-merge-conflict-bot'] nobody
156-67405
5 months ago
156-67406
156 days ago
6-5823
6 days
27003 eric-wieser
author:eric-wieser
chore: use `Simp.ResultQ` more often Also uses `~q` in place of manual `isDefEq` matching. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-meta 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
154-82029
5 months ago
154-82030
154 days ago
32-67299
32 days
28622 alreadydone
author:alreadydone
chore(Mathlib): replace `=>` by `↦` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
148-40305
4 months ago
148-40306
148 days ago
0-55389
15 hours
28626 alreadydone
author:alreadydone
chore(Archive, Counterexamples): replace => by ↦ --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
146-69431
4 months ago
146-69432
146 days ago
2-46227
2 days
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-data new-contributor 24/26 Mathlib/Data/TypeVec.lean 1 7 ['Equilibris', 'alexkeizer', 'github-actions', 'mathlib4-merge-conflict-bot'] nobody
145-36747
4 months ago
145-36748
145 days ago
13-47613
13 days
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) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict new-contributor 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
145-16067
4 months ago
167-78389
167 days ago
7-51497
7 days
28042 kckennylau
author:kckennylau
feat(Topology/ValuativeRel): a topological basis indexed by pairs of elements --- The pullback PR of #27314 and #27163. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-ring-theory 140/23 Mathlib/RingTheory/Valuation/ValuativeRel.lean,Mathlib/Topology/Algebra/Valued/ValuativeRel.lean 2 3 ['github-actions', 'grunweg', 'mathlib4-merge-conflict-bot'] nobody
145-16021
4 months ago
154-67465
154 days ago
7-2766
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict new-contributor 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
144-64299
4 months ago
167-78390
167 days ago
7-53541
7 days
27785 staroperator
author:staroperator
chore(Algebra/Group/Submonoid): golf `Nat.addSubmonoidClosure_one` using `simp` This should improve the proof readability. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra large-import
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
140-21362
4 months ago
140-21363
140 days ago
26-29321
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] ``` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-meta 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
140-21233
4 months ago
140-21234
140 days ago
12-66568
12 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? [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-data large-import 220/3 Mathlib/Data/Real/Embedding.lean 1 2 ['github-actions', 'mathlib4-merge-conflict-bot'] nobody
131-14352
4 months ago
131-14353
131 days ago
40-31514
40 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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-category-theory 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
128-67579
4 months ago
128-67580
128 days ago
0-1045
17 minutes
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 --- merge-conflict t-logic new-contributor 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
127-70330
4 months ago
127-70331
127 days ago
10-49648
10 days
27933 grunweg
author:grunweg
chore(OrdNode): format code example in code blocks Wrap them in code blocks (and unindent them; that indentation is not needed any more). This also avoids warnings from the linter in #27898. ------- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-data 459/212 Mathlib/Data/Ordmap/Ordnode.lean 1 4 ['eric-wieser', 'github-actions', 'grunweg', 'mathlib4-merge-conflict-bot'] nobody
124-20963
4 months ago
124-20964
124 days ago
39-68381
39 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 merge-conflict t-topology 651/0 Mathlib.lean,Mathlib/Topology/Algebra/FilterBasis.lean,Mathlib/Topology/Algebra/FilterBasisNew.lean,Mathlib/Topology/Algebra/Nonarchimedean/Bases.lean,Mathlib/Topology/Algebra/Nonarchimedean/BasesNew.lean 5 3 ['ADedecker', 'github-actions', 'mathlib4-merge-conflict-bot'] PatrickMassot
assignee:PatrickMassot
121-82574
3 months ago
121-82575
121 days ago
87-78694
87 days
29330 plp127
author:plp127
chore: define `Fin.cycleIcc` with conditions Redefine `Fin.cycleIcc` using conditionals instead of composing existing `Fin` operations together. Its worst-case runtime drops from O(n) to O(1). As a bonus, the definition no longer needs explaining. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-group-theory 61/68 Mathlib/GroupTheory/Perm/Fin.lean 1 10 ['JovanGerb', 'eric-wieser', 'github-actions', 'mathlib4-merge-conflict-bot', 'plp127', 'tb65536'] nobody
113-7771
3 months ago
113-7772
113 days ago
19-72402
19 days
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-category-theory 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
107-59363
3 months ago
107-59364
107 days ago
0-4044
1 hour
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebraic-topology t-category-theory 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
106-78765
3 months ago
201-86049
201 days ago
0-1046
17 minutes
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
98-85634
3 months ago
98-85635
98 days ago
25-73895
25 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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-ring-theory 172/0 Counterexamples.lean,Counterexamples/DiscreteTopologyWithNontrivialValuation.lean 2 14 ['github-actions', 'grunweg', 'kckennylau', 'mathlib4-merge-conflict-bot', 'pechersky'] nobody
94-65836
3 months ago
94-65837
94 days ago
67-78029
67 days
25978 Bergschaf
author:Bergschaf
feat(Order/Sublocale): Open Sublocales --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) - [x] depends on: #25089 merge-conflict t-order 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
83-54692
2 months ago
156-12569
156 days ago
0-1326
22 minutes
28132 dupuisf
author:dupuisf
feat: preliminary `grind` tags for `IsUnit` This PR adds preliminary `grind` tags for the `IsUnit` predicate. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra
label:t-algebra$
61/17 Mathlib/Algebra/Group/Action/Units.lean,Mathlib/Algebra/Group/Units/Defs.lean,Mathlib/Algebra/GroupWithZero/Units/Basic.lean,Mathlib/Algebra/Ring/Units.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Order.lean,Mathlib/Analysis/SpecialFunctions/ContinuousFunctionalCalculus/Rpow/Basic.lean 6 3 ['github-actions', 'mathlib4-merge-conflict-bot'] kim-em
assignee:kim-em
71-42435
2 months ago
71-42436
71 days ago
80-71574
80 days
26827 pechersky
author:pechersky
feat(Analysis/Normed/ValuativeRel): helper instance for NormedField --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) - [x] depends on: #26713 - [x] depends on: #26826 merge-conflict t-algebra t-number-theory t-analysis
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
63-71039
2 months ago
63-71039
63 days ago
126-50240
126 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. merge-conflict t-data 35/0 Mathlib/Data/List/Scan.lean 1 11 ['ShreckYe', 'github-actions', 'mathlib4-merge-conflict-bot', 'themathqueen', 'vlad902'] pechersky
assignee:pechersky
63-27270
2 months ago
66-25001
66 days ago
74-48754
74 days
26240 grunweg
author:grunweg
perf(CommandLinterLinter): use Substring more Probably, these changes make little difference, but let's find out. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-linter RFC 14/15 Mathlib/Tactic/Linter/CommandStart.lean 1 6 ['github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'mathlib4-merge-conflict-bot'] joneugster
assignee:joneugster
57-78316
1 month ago
57-78317
57 days ago
150-49908
150 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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict CI 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
57-57263
1 month ago
72-20745
72 days ago
41-46786
41 days
24850 pechersky
author:pechersky
feat(Topology/UniformSpace/Ultra): uniform spaces induced by pseudometrics are ultra if system is ultra Any uniform space has a natural system of pseudometrics definable on it, comprised of those pseudometrics constructed from a descending chain of equivalence relation entourages. In a nonarchimedean uniformity, this pseudometric system induces the uniformity. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) - [x] depends on: #23111 merge-conflict t-topology 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
57-7126
1 month ago
57-7127
57 days ago
162-10999
162 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 merge-conflict t-topology large-import 174/5 Mathlib/Topology/Compactness/CompactlyCoherentSpace.lean 1 5 ['github-actions', 'joelriou', 'mathlib4-merge-conflict-bot', 'scholzhannah'] ADedecker
assignee:ADedecker
57-6958
1 month ago
57-6959
57 days ago
147-61529
147 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`) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-data 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
57-6604
1 month ago
57-6605
57 days ago
133-15886
133 days
27534 PierreQuinton
author:PierreQuinton
feat: a typeclass for `sSup`/`sInf` to be lawful Adds lawful infima and suprema type classes. A preorder with lawful suprema: whenever a set has a least upper bound, `sSup` returns a least upper bound for that set. A preorder with lawful infima: whenever a set has a greatest lower bound, `sInf` returns a greastest lower bound for that set. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-order 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
57-6441
1 month ago
57-6442
57 days ago
114-33795
114 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. merge-conflict t-combinatorics new-contributor 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
57-6299
1 month ago
57-6300
57 days ago
99-48372
99 days
28871 JaafarTanoukhi
author:JaafarTanoukhi
feat(Combinatorics/Digraph): Tournaments Define orientations and tournaments. Related to #26771. Co-authored-by: Rida Hamadani --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-combinatorics new-contributor 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
57-6146
1 month ago
57-6147
57 days ago
71-35799
71 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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-data 35/0 Mathlib/Data/Multiset/Fintype.lean 1 9 ['Ruben-VandeVelde', 'github-actions', 'llllvvuu', 'mathlib4-merge-conflict-bot', 'vihdzp', 'wwylele'] pechersky
assignee:pechersky
57-6108
1 month ago
57-6109
57 days ago
69-16483
69 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) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-combinatorics new-contributor 476/0 Mathlib.lean,Mathlib/Combinatorics/Digraph/Maps.lean 2 2 ['github-actions', 'mathlib4-merge-conflict-bot'] awainverse
assignee:awainverse
57-5512
1 month ago
57-5513
57 days ago
54-81855
54 days
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]`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-data 41/0 Mathlib.lean,Mathlib/Data/FunLike/Graded.lean 2 2 ['github-actions', 'mathlib4-merge-conflict-bot'] nobody
57-5324
1 month ago
57-5325
57 days ago
40-71592
40 days
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 -/ ``` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-meta 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
57-533
1 month ago
57-534
57 days ago
11-59965
11 days
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-combinatorics 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
56-65194
1 month ago
57-6624
57 days ago
137-24962
137 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` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-data 2/3 Mathlib/Data/Fin/Embedding.lean 1 2 ['github-actions', 'mathlib4-merge-conflict-bot'] nobody
56-64970
1 month ago
115-74869
115 days ago
18-35802
18 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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) I found this being not-simp frustrating when talking about submodules over a valuation subring. merge-conflict t-algebra
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 26 ['artie2000', 'eric-wieser', 'github-actions', 'j-loreaux', 'kckennylau', 'leanprover-bot', 'leanprover-radar', 'linesthatinterlace', 'mathlib4-merge-conflict-bot', 'pechersky'] joelriou
assignee:joelriou
30-38311
30 days ago
51-74260
51 days ago
60-49993
60 days
33020 FormulaRabbit81
author:FormulaRabbit81
chore(Topology): Deprecate file --- - [ ] depends on: #30851 deprecation [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology large-import merge-conflict 82/49 Mathlib/Topology/Compactness/HilbertCubeEmbedding.lean,Mathlib/Topology/MetricSpace/HausdorffAlexandroff.lean,Mathlib/Topology/MetricSpace/PiNat.lean 3 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
28-18404
28 days ago
28-18405
28 days ago
0-13670
3 hours
32918 michelsol
author:michelsol
feat: define `supEdist` and `supDist` Create a new file Topology.MetricSpace.SupDistance and define the supremal distance in (extended) metric spaces. The defined `supEdist` and `supDist` will have similar theory to the already existing `infEdist` and `infDist`. The motivation is to be able to define the radius of a minimal bounding sphere as the infimum of the supDist later. [zulip discussion here](https://leanprover.zulipchat.com/#narrow/channel/116395-maths/topic/Formalizing.20Jung's.20theorem.20and.20minimal.20bounding.20spheres) t-topology new-contributor merge-conflict 75/0 Mathlib.lean,Mathlib/Topology/MetricSpace/SupDistance.lean 2 2 ['github-actions', 'mathlib4-merge-conflict-bot'] RemyDegenne
assignee:RemyDegenne
9-48692
9 days ago
9-48694
9 days ago
21-957
21 days
31754 dagurtomas
author:dagurtomas
feat(Topology/Category): light profinite sets are injective objects From [LeanCondensed](https://github.com/dagurtomas/LeanCondensed) --- - [ ] depends on: #32660 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology t-category-theory merge-conflict 304/0 Mathlib.lean,Mathlib/Topology/Category/LightProfinite/Injective.lean,Mathlib/Topology/Separation/Profinite.lean 3 4 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
7-48448
7 days ago
7-48449
7 days ago
1-8608
1 day
33561 kbuzzard
author:kbuzzard
chore: cont -> continuous_toFun This field is sometimes called `cont` and sometimes `continuous_toFun`. I noticed that the `continuity` tactic sometimes takes a lot longer to prove `cont` even if `continuous_toFun` is available so I thought I'd change them all to see if this speed up mathlib. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict 171/149 Mathlib/Algebra/Category/ContinuousCohomology/Basic.lean,Mathlib/Algebra/Category/ModuleCat/Topology/Homology.lean,Mathlib/Analysis/Analytic/Composition.lean,Mathlib/Analysis/Analytic/Polynomial.lean,Mathlib/Analysis/CStarAlgebra/CStarMatrix.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/NonUnital.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Unital.lean,Mathlib/Analysis/Calculus/ContDiff/FaaDiBruno.lean,Mathlib/Analysis/Calculus/FDeriv/Basic.lean,Mathlib/Analysis/Calculus/FDeriv/Extend.lean,Mathlib/Analysis/Distribution/ContDiffMapSupportedIn.lean,Mathlib/Analysis/Distribution/DerivNotation.lean,Mathlib/Analysis/Distribution/SchwartzSpace.lean,Mathlib/Analysis/Distribution/TemperedDistribution.lean,Mathlib/Analysis/Distribution/TestFunction.lean,Mathlib/Analysis/Fourier/FourierTransform.lean,Mathlib/Analysis/Fourier/LpSpace.lean,Mathlib/Analysis/InnerProductSpace/LinearPMap.lean,Mathlib/Analysis/LocallyConvex/Barrelled.lean,Mathlib/Analysis/LocallyConvex/PointwiseConvergence.lean,Mathlib/Analysis/LocallyConvex/Separation.lean,Mathlib/Analysis/LocallyConvex/WeakOperatorTopology.lean,Mathlib/Analysis/LocallyConvex/WeakSpace.lean,Mathlib/Analysis/Normed/Affine/Isometry.lean,Mathlib/Analysis/Normed/Algebra/Spectrum.lean,Mathlib/Analysis/Normed/Lp/PiLp.lean,Mathlib/Analysis/Normed/Lp/ProdLp.lean,Mathlib/Analysis/Normed/Lp/lpSpace.lean,Mathlib/Analysis/Normed/Module/Alternating/Basic.lean,Mathlib/Analysis/Normed/Module/Multilinear/Basic.lean,Mathlib/Analysis/Normed/Module/WeakDual.lean,Mathlib/Analysis/Normed/Operator/Banach.lean,Mathlib/Analysis/Normed/Operator/BoundedLinearMaps.lean,Mathlib/Analysis/Normed/Operator/Extend.lean,Mathlib/Analysis/RCLike/Extend.lean,Mathlib/Geometry/Euclidean/Incenter.lean,Mathlib/Geometry/Manifold/LocalDiffeomorph.lean,Mathlib/Geometry/Manifold/MFDeriv/Atlas.lean,Mathlib/MeasureTheory/Function/ConditionalExpectation/Basic.lean,Mathlib/MeasureTheory/Function/ConditionalExpectation/CondexpL1.lean,Mathlib/MeasureTheory/Function/SimpleFuncDenseLp.lean,Mathlib/MeasureTheory/Integral/Bochner/L1.lean,Mathlib/MeasureTheory/Measure/FiniteMeasure.lean,Mathlib/NumberTheory/ModularForms/JacobiTheta/TwoVariable.lean,Mathlib/Probability/Distributions/Fernique.lean,Mathlib/Probability/Moments/CovarianceBilinDual.lean,Mathlib/Topology/Algebra/AffineSubspace.lean,Mathlib/Topology/Algebra/Algebra.lean,Mathlib/Topology/Algebra/ContinuousAffineEquiv.lean,Mathlib/Topology/Algebra/ContinuousAffineMap.lean,Mathlib/Topology/Algebra/Module/Alternating/Basic.lean,Mathlib/Topology/Algebra/Module/Alternating/Topology.lean,Mathlib/Topology/Algebra/Module/CharacterSpace.lean,Mathlib/Topology/Algebra/Module/Equiv.lean,Mathlib/Topology/Algebra/Module/LinearMap.lean,Mathlib/Topology/Algebra/Module/LinearMapPiProd.lean,Mathlib/Topology/Algebra/Module/Multilinear/Basic.lean,Mathlib/Topology/Algebra/Module/Multilinear/Topology.lean,Mathlib/Topology/Algebra/Module/PointwiseConvergence.lean,Mathlib/Topology/Algebra/Module/Star.lean,Mathlib/Topology/Algebra/Module/StrongTopology.lean,Mathlib/Topology/Algebra/Module/WeakDual.lean,Mathlib/Topology/ContinuousMap/Algebra.lean,Mathlib/Topology/ContinuousMap/Ideals.lean,Mathlib/Topology/Instances/TrivSqZeroExt.lean,Mathlib/Topology/VectorBundle/Basic.lean 66 5 ['eric-wieser', 'github-actions', 'kbuzzard', 'leanprover-radar', 'mathlib4-merge-conflict-bot'] nobody
7-40386
7 days ago
7-40387
7 days ago
2-79879
2 days
33330 michael-novak-math
author:michael-novak-math
feat: add arc-length reparametrization of parametrized curves add new definitions of arc-length reparametrization and its corresponding parameter transformation and a theorem establishing the desired properties. t-analysis new-contributor merge-conflict 311/0 Mathlib.lean,Mathlib/Analysis/Calculus/ArcLengthReparametrization.lean,Mathlib/MeasureTheory/Integral/IntervalIntegral/FundThmCalculus.lean,docs/references.bib,lake-manifest.json 5 53 ['SnirBroshi', 'github-actions', 'grunweg', 'j-loreaux', 'mathlib4-merge-conflict-bot', 'michael-novak-math'] j-loreaux
assignee:j-loreaux
7-30246
7 days ago
7-30247
7 days ago
6-57754
6 days
30855 Ruben-VandeVelde
author:Ruben-VandeVelde
fix: deprecate IsTotal in favour of Std.Total --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order merge-conflict RFC 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'] nobody
6-69843
6 days ago
57-76165
57 days ago
24-78190
24 days
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict large-import t-logic 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
6-67632
6 days ago
144-45585
144 days ago
3-938
3 days
31595 astrainfinita
author:astrainfinita
chore: redefine `Ideal.IsPrime` Redefine `Ideal.IsPrime` to make it correct for non-commutative cases --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict
label:t-algebra$
330/100 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/Ideal/Quotient/Operations.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 22 29 ['alreadydone', 'artie2000', 'astrainfinita', 'erdOne', 'github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'mathlib4-merge-conflict-bot'] alreadydone
assignee:alreadydone
2-76800
2 days ago
4-48894
4 days ago
28-50719
28 days
33435 astrainfinita
author:astrainfinita
feat: algebra automorphisms of monoid algebras --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra
label:t-algebra$
53/3 Mathlib/Algebra/MonoidAlgebra/Basic.lean 1 2 ['github-actions', 'mathlib4-merge-conflict-bot'] kbuzzard
assignee:kbuzzard
1-50299
1 day ago
1-50300
1 day ago
13-11452
13 days
33870 jcommelin
author:jcommelin
feat(Data/Matrix/Cartan): add IsSymm lemmas and simplify IsSimplyLaced proofs This PR adds symmetry theorems for A, D, and E-series Cartan matrices, a DecidablePred instance for IsSimplyLaced, and a lemma reducing simply-laced checks to half the entries for symmetric matrices. The E-series and F₄/G₂ proofs are simplified to use decide. --- - [x] depends on: #33538 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data merge-conflict 37/8 Mathlib/Data/Matrix/Cartan.lean 1 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
1-40253
1 day ago
1-43851
1 day ago
0-13862
3 hours
33930 chrisflav
author:chrisflav
feat(AlgebraicGeometry): gluing colimits in `P.Over ⊤ S` Let `D : J ⥤ P.Over ⊤ S` be a diagram and `𝒰` a locally directed open cover of `S` (e.g., the cover of all affine opens of `S`). Suppose the restrictions of `D` to `Dᵢ : J ⥤ P.Over ⊤ (𝒰.X i)` have a colimit for every `i`, then we show that also `D` has a colimit under suitable assumptions. This can be used to reduce existence of certain colimits in `P.Over ⊤ S` to the case where `S` is affine. From Pi1. --- - [ ] depends on: #33898 - [ ] depends on: #33932 - [ ] depends on: #33931 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebraic-geometry 578/11 Mathlib.lean,Mathlib/AlgebraicGeometry/ColimitsOver.lean,Mathlib/AlgebraicGeometry/Cover/Directed.lean,Mathlib/AlgebraicGeometry/Gluing.lean,Mathlib/AlgebraicGeometry/RelativeGluing.lean,Mathlib/CategoryTheory/MorphismProperty/Composition.lean,Mathlib/CategoryTheory/MorphismProperty/OverAdjunction.lean 7 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
0-56273
15 hours ago
unknown
unknown

Stale new contributor PRs

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
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)` [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-algebra new-contributor
label:t-algebra$
5/0 Mathlib/Algebra/Group/Basic.lean 1 3 ['eric-wieser', 'github-actions', 'kim-em'] nobody
517-84096
1 year ago
unknown
unknown
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`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-data new-contributor 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
513-69005
1 year ago
unknown
unknown
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`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-data new-contributor 90/0 Mathlib/Data/Nat/PartENat.lean 1 3 ['erdOne', 'github-actions', 'urkud'] nobody
500-80895
1 year ago
unknown
unknown
15121 Eloitor
author:Eloitor
feat: iff theorems for IsSplitEpi and IsSplitMono in opposite category --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-category-theory new-contributor 40/0 Mathlib/CategoryTheory/EpiMono.lean 1 3 ['github-actions', 'joelriou', 'mattrobball'] nobody
500-43840
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra blocked-by-other-PR new-contributor
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
477-54899
1 year ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR new-contributor t-logic 300/7 Mathlib/ModelTheory/Complexity.lean,Mathlib/ModelTheory/Equivalence.lean,Mathlib/ModelTheory/Syntax.lean 3 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
469-50877
1 year ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR new-contributor t-logic 415/7 Mathlib/ModelTheory/Complexity.lean,Mathlib/ModelTheory/Equivalence.lean,Mathlib/ModelTheory/Syntax.lean 3 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
469-50877
1 year ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR new-contributor t-logic 525/7 Mathlib/ModelTheory/Complexity.lean,Mathlib/ModelTheory/Equivalence.lean,Mathlib/ModelTheory/Syntax.lean 3 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
469-50876
1 year ago
unknown
unknown
14619 Command-Master
author:Command-Master
chore: Merge `Trunc` to `Squash` Remove `Trunc` and use `Squash` instead --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP new-contributor 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
460-11027
1 year ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR t-data new-contributor merge-conflict awaiting-author 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
451-73534
1 year ago
unknown
unknown
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`? [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-combinatorics new-contributor 24/0 Mathlib/Combinatorics/SimpleGraph/Map/Finite.lean 1 11 ['awueth', 'github-actions', 'jcommelin', 'kim-em', 'urkud'] nobody
449-62842
1 year ago
unknown
unknown
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. please-adopt t-data new-contributor merge-conflict 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
441-44844
1 year ago
unknown
unknown
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]`. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra t-order new-contributor
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
435-15410
1 year ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author new-contributor t-logic 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
432-57931
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) merge-conflict awaiting-author new-contributor t-logic 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
428-10363
1 year ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra new-contributor
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
398-32780
1 year ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-topology new-contributor 27/0 Mathlib/Topology/Order/DenselyOrdered.lean 1 8 ['github-actions', 'vihdzp'] nobody
364-54792
11 months ago
unknown
unknown
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 merge-conflict awaiting-author t-combinatorics new-contributor 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
363-73878
11 months ago
unknown
unknown
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 merge-conflict blocked-by-other-PR t-combinatorics new-contributor 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
363-73878
11 months ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-computability awaiting-author new-contributor 186/0 Mathlib.lean,Mathlib/Computability/Timed/InsertionSort.lean,Mathlib/Computability/Timed/Merge.lean 3 2 ['github-actions', 'trivial1711'] nobody
363-39797
11 months ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-algebra new-contributor
label:t-algebra$
78/0 Mathlib/Algebra/Group/Defs.lean 1 13 ['github-actions', 'hannahfechtner', 'jcommelin', 'kbuzzard', 'kim-em', 'trivial1711'] nobody
360-977
11 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-algebra new-contributor
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
358-61456
11 months ago
unknown
unknown
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`) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-measure-probability new-contributor 203/40 Mathlib/MeasureTheory/Function/LpSeminorm/CompareExp.lean,Mathlib/MeasureTheory/Function/LpSpace.lean 2 1 ['github-actions'] nobody
351-78804
11 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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR large-import new-contributor merge-conflict awaiting-author t-topology 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
339-36114
11 months ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-computability awaiting-author new-contributor 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
334-70213
11 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-algebra new-contributor
label:t-algebra$
43/0 Mathlib/Algebra/BigOperators/Group/Finset/Basic.lean 1 1 ['github-actions', 'j-loreaux'] nobody
329-38984
10 months ago
unknown
unknown
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) ``` merge-conflict t-algebra t-category-theory new-contributor
label:t-algebra$
47/8 Mathlib/RepresentationTheory/FDRep.lean 1 19 ['github-actions', 'grhkm21', 'joelriou', 'kim-em', 'mathlib-bors'] nobody
320-78811
10 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR new-contributor t-logic 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
317-21235
10 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-topology new-contributor 285/1 Mathlib.lean,Mathlib/Topology/ContinuousMap/MvPolynomial.lean,Mathlib/Topology/ContinuousMap/StoneWeierstrass.lean 3 1 ['github-actions'] nobody
315-64825
10 months ago
unknown
unknown
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`. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-analysis new-contributor 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
307-60651
10 months ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data enhancement new-contributor merge-conflict awaiting-author 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 17 ['chrisflav', 'eric-wieser', 'github-actions', 'j-loreaux', 'markimunro'] nobody
289-9650
9 months ago
unknown
unknown
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 t-measure-probability new-contributor merge-conflict awaiting-author t-analysis 60/1 Mathlib/MeasureTheory/Integral/FundThmCalculus.lean 1 3 ['github-actions', 'hrmacbeth', 'victorliu5296'] nobody
284-4639
9 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-analysis new-contributor 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
280-76959
9 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-category-theory new-contributor 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
280-73227
9 months ago
unknown
unknown
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-topology new-contributor 281/1 Mathlib.lean,Mathlib/Topology/Covering/Basic.lean,Mathlib/Topology/Covering/Lift.lean 3 9 ['alreadydone', 'github-actions', 'grunweg', 'vbeffara'] nobody
279-75955
9 months ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-analysis new-contributor 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
272-47153
8 months ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-algebra new-contributor
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
272-43285
8 months ago
unknown
unknown
23791 SEU-Prime
author:SEU-Prime
Create AmiceTrans.lean --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-number-theory new-contributor 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
260-16897
8 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-algebra t-category-theory new-contributor
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
257-7724
8 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR new-contributor t-computability merge-conflict awaiting-zulip 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
254-40403
8 months ago
unknown
unknown
24008 meithecatte
author:meithecatte
chore(EpsilonNFA): replace manual lemmas with @[simps] --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-computability awaiting-author new-contributor 2/24 Mathlib/Computability/EpsilonNFA.lean 1 2 ['YaelDillies', 'github-actions', 'urkud'] nobody
248-85982
8 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-topology large-import new-contributor 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
232-58323
7 months ago
unknown
unknown
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`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) please-adopt t-algebra new-contributor merge-conflict awaiting-author
label:t-algebra$
78/0 Mathlib/LinearAlgebra/UnitaryGroup.lean 1 8 ['chrisflav', 'jcommelin', 'leanprover-community-bot-assistant'] nobody
222-30276
7 months ago
unknown
unknown
23929 meithecatte
author:meithecatte
feat(Computability/NFA): improve bound on pumping lemma --- - [x] depends on: #25321 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-computability awaiting-zulip 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
221-50005
7 months ago
221-50006
221 days ago
0-37135
10 hours
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author new-contributor t-meta 171/48 Mathlib/Tactic/Polyrith.lean,scripts/polyrith_sage.py 2 16 ['eric-wieser', 'github-actions', 'hanwenzhu', 'kim-em', 'miguelmarco', 'mkoeppe'] nobody
215-22829
7 months ago
unknown
unknown
25218 kckennylau
author:kckennylau
feat(AlgebraicGeometry): Tate normal form of elliptic curves --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebraic-geometry awaiting-zulip new-contributor 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
194-19590
6 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra new-contributor
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
194-19586
6 months ago
unknown
unknown
10541 xgenereux
author:xgenereux
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-algebra new-contributor
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', 'YaelDillies', 'eric-wieser', 'fpvandoorn', 'github-actions', 'mariainesdff', 'mathlib4-dependent-issues-bot', 'mattrobball', 'xgenereux'] AntoineChambert-Loir
assignee:AntoineChambert-Loir
189-75068
6 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-topology new-contributor 63/0 Mathlib/Topology/MetricSpace/HausdorffDimension.lean 1 10 ['AntoineChambert-Loir', 'FrankieNC', 'github-actions', 'grunweg'] nobody
185-48292
6 months ago
185-62703
185 days ago
0-12255
3 hours
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` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebraic-topology WIP t-category-theory new-contributor merge-conflict 720/0 Mathlib.lean,Mathlib/AlgebraicTopology/AugmentedSimplexCategory.lean,Mathlib/AlgebraicTopology/SimplicialObject.lean,Mathlib/Order/Category/FinLinOrd.lean 4 5 ['TwoFX', 'YaelDillies', 'joelriou', 'jstoobysmith'] nobody
167-78130
5 months ago
unknown
unknown
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` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) - [ ] depends on: #25483 - [ ] depends on: #25485 merge-conflict t-set-theory blocked-by-other-PR new-contributor 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
163-84355
5 months ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) - [ ] depend on: #25483 merge-conflict t-set-theory new-contributor 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
163-84351
5 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) - [ ] depends on: #25483 merge-conflict t-set-theory blocked-by-other-PR new-contributor 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
163-84346
5 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-meta new-contributor 17/5 Mathlib/Tactic/ComputeDegree.lean,MathlibTest/ComputeDegree.lean 2 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
163-84321
5 months ago
unknown
unknown
18646 jxjwan
author:jxjwan
feat(RingTheory): isotypic components --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-ring-theory new-contributor 308/0 Mathlib/Order/CompactlyGenerated/Basic.lean,Mathlib/RingTheory/Isotypic.lean,Mathlib/RingTheory/SimpleModule.lean 3 1 ['github-actions'] nobody
162-86342
5 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-number-theory new-contributor large-import 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
158-3483
5 months ago
unknown
unknown
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 awaiting-author t-combinatorics new-contributor 14/0 Mathlib/Combinatorics/SimpleGraph/Subgraph.lean 1 3 ['b-mehta', 'github-actions', 'xcloudyunx'] b-mehta
assignee:b-mehta
156-19229
5 months ago
156-33309
156 days ago
25-82865
25 days
22925 ggranberry
author:ggranberry
feat(Mathlib/PlaceHolder/ToeplitzHausdorff): Toeplitz-Hausdorff --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP new-contributor will-close-soon awaiting-author help-wanted t-analysis 411/0 Mathlib/PlaceHolder/ToeplitzHausdorff.lean,Mathlib/PlaceHolder/ToeplitzHausdorff_v2.lean 2 11 ['faenuccio', 'ggranberry', 'github-actions'] faenuccio
assignee:faenuccio
154-81753
5 months ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-data new-contributor 103/0 Mathlib/Data/Set/Prod.lean,Mathlib/SetTheory/ZFC/Basic.lean 2 10 ['Ruben-VandeVelde', 'VTrelat', 'github-actions', 'leanprover-community-bot-assistant'] nobody
154-71673
5 months ago
unknown
unknown
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. --- please-adopt new-contributor merge-conflict modifies-tactic-syntax good first issue t-meta 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
153-741
5 months ago
unknown
unknown
20722 ctchou
author:ctchou
feat(Counterexamples): the Vitali set is non-measurable --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) please-adopt t-measure-probability new-contributor merge-conflict 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
151-79567
4 months ago
unknown
unknown
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 blocked-by-other-PR new-contributor merge-conflict awaiting-author t-logic 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
149-14979
4 months ago
152-508
152 days ago
0-32456
9 hours
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra blocked-by-other-PR new-contributor
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
146-51487
4 months ago
unknown
unknown
28095 Equilibris
author:Equilibris
Univ generic corec Draft PR: Adding variable universe corecursor for PFunctor --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict new-contributor 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
145-36749
4 months ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-data new-contributor 24/26 Mathlib/Data/TypeVec.lean 1 7 ['Equilibris', 'alexkeizer', 'github-actions', 'mathlib4-merge-conflict-bot'] nobody
145-36748
4 months ago
145-36749
145 days ago
13-47613
13 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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) - [ ] depends on: #25483 - [ ] depends on: #25485 - [ ] depends on: #25486 merge-conflict t-set-theory blocked-by-other-PR new-contributor 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
145-16105
4 months ago
unknown
unknown
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) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict new-contributor 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
145-16068
4 months ago
167-78390
167 days ago
7-51497
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict new-contributor 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
144-64300
4 months ago
167-78391
167 days ago
7-53541
7 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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-data new-contributor 326/0 Mathlib/Data/Nat/Choose/AbelBinomial.lean 1 28 ['ElifUskuplu', 'FrankieNC', 'github-actions', 'iu-isgood'] nobody
144-64061
4 months ago
unknown
unknown
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data new-contributor 16/21 Mathlib/Data/PFunctor/Multivariate/W.lean 1 8 ['Equilibris', 'alexkeizer', 'github-actions'] nobody
136-49270
4 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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR new-contributor merge-conflict awaiting-author t-analysis 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
136-47890
4 months ago
unknown
unknown
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! [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-algebra new-contributor
label:t-algebra$
10/0 Mathlib/LinearAlgebra/Projection.lean 1 7 ['PSchwahn', 'github-actions', 'joelriou', 'kckennylau'] joelriou
assignee:joelriou
128-35429
4 months ago
128-66532
128 days ago
73-38219
73 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 --- merge-conflict t-logic new-contributor 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
127-70331
4 months ago
127-70332
127 days ago
10-49648
10 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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-differential-geometry new-contributor 36/0 Mathlib/Geometry/Manifold/ContMDiff/Defs.lean 1 13 ['bwangpj', 'girving', 'github-actions', 'grunweg', 'kbuzzard', 'sgouezel'] sgouezel
assignee:sgouezel
127-50184
4 months ago
128-4219
128 days ago
22-76960
22 days
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-measure-probability new-contributor 8/0 Mathlib/MeasureTheory/Integral/Bochner/Set.lean 1 6 ['RemyDegenne', 'github-actions', 'sgouezel', 'thefundamentaltheor3m'] nobody
125-66053
4 months ago
216-73891
216 days ago
0-7890
2 hours
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. awaiting-author t-analysis new-contributor 383/0 Mathlib/Analysis/Complex/Residue/Basic.lean 1 17 ['Periecle', 'github-actions', 'hrmacbeth', 'llllvvuu', 'loefflerd'] nobody
112-69531
3 months ago
unknown
unknown
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-category-theory new-contributor 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
111-70362
3 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author new-contributor t-measure-probability 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
108-42430
3 months ago
139-255
139 days ago
0-22659
6 hours
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-category-theory new-contributor 17/0 Mathlib/CategoryTheory/Limits/Shapes/Products.lean 1 6 ['chrisflav', 'github-actions', 'leanprover-community-bot-assistant', 'ppls-nd-prs', 'robin-carlier'] nobody
107-84575
3 months ago
209-7575
209 days ago
0-45487
12 hours
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) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) IMO awaiting-author new-contributor 196/0 Archive.lean,Archive/Imo/Imo1975Q3.lean 2 36 ['Antidite', 'LLaurance', 'github-actions', 'jsm28'] jsm28
assignee:jsm28
102-50321
3 months ago
102-50321
102 days ago
46-21614
46 days
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] --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR new-contributor 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
96-64841
3 months ago
unknown
unknown
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 merge-conflict t-category-theory new-contributor 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
96-60776
3 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author new-contributor t-measure-probability 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
96-59626
3 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebraic-topology blocked-by-other-PR new-contributor 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
88-53957
2 months ago
158-64493
158 days ago
0-2143
35 minutes
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-group-theory new-contributor 6/0 Mathlib/GroupTheory/GroupAction/CardCommute.lean 1 17 ['github-actions', 'kckennylau', 'plp127', 'tb65536'] tb65536
assignee:tb65536
86-69876
2 months ago
86-69876
86 days ago
8-4679
8 days
25225 xcloudyunx
author:xcloudyunx
feat(Combinatorics/SimpleGraph): Eulerian walk in connected graph contains all vertices --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-combinatorics new-contributor 16/0 Mathlib/Combinatorics/SimpleGraph/Trails.lean 1 6 ['IvanRenison', 'github-actions', 'vlad902'] kmill
assignee:kmill
85-33408
2 months ago
unknown
unknown
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`). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
83-56840
2 months ago
unknown
unknown
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! [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-number-theory new-contributor large-import 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
79-2879
2 months ago
94-63955
94 days ago
47-56535
47 days
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor merge-conflict file-removed awaiting-author t-topology 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
78-81009
2 months ago
99-63638
99 days ago
0-553
9 minutes
30303 franv314
author:franv314
chore(Topology/Instances): add deprecated module Add deprecated module to moved Cantor set file. --- - [ ] depends on: #30299 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR new-contributor 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
78-81007
2 months ago
99-61839
99 days ago
0-8
8 seconds
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-algebra new-contributor
label:t-algebra$
47/0 Mathlib/Algebra/Group/Subgroup/Pointwise.lean 1 10 ['FrederickPu', 'eric-wieser', 'github-actions', 'plp127', 'tb65536'] nobody
78-69838
2 months ago
87-59872
87 days ago
0-40723
11 hours
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`. --- --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-algebra new-contributor
label:t-algebra$
94/0 Mathlib/LinearAlgebra/Matrix/Transvection.lean,MathlibTest/matrix.lean 2 3 ['github-actions', 'riccardobrasca', 'zach1502'] nobody
72-80530
2 months ago
72-80530
72 days ago
41-49475
41 days
22361 rudynicolop
author:rudynicolop
feat(Computability/NFA): nfa closure properties Add the closure properties union, intersection and reversal for NFA. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-computability merge-conflict awaiting-author awaiting-zulip 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
72-22135
2 months ago
unknown
unknown
30158 nicolaviolette
author:nicolaviolette
feat: combinatorics simplegraph basic --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-combinatorics new-contributor 9/4 Mathlib/Combinatorics/SimpleGraph/Basic.lean 1 3 ['b-mehta', 'github-actions'] b-mehta
assignee:b-mehta
72-13660
2 months ago
72-13660
72 days ago
31-68997
31 days
27229 WilliamCoram
author:WilliamCoram
feat(GroupTheory/DoubleCoset): multiple lemmas From FLT --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) FLT t-group-theory 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
71-68559
2 months ago
84-85290
84 days ago
92-33213
92 days
26901 5hv5hvnk
author:5hv5hvnk
feat: a simproc version of `compute_degree` Wrap `compute_degree` in a simproc for use by simp. Closes #22219. --- awaiting-CI new-contributor merge-conflict awaiting-author t-meta 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
69-60328
2 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-ring-theory new-contributor 17/0 Mathlib/RingTheory/MvPolynomial/Homogeneous.lean 1 6 ['LiamSchilling', 'chrisflav', 'github-actions'] chrisflav
assignee:chrisflav
63-27376
2 months ago
113-84317
113 days ago
2-17024
2 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` [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory large-import new-contributor merge-conflict awaiting-zulip t-meta 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
63-23319
2 months ago
103-1985
103 days ago
0-29227
8 hours
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR large-import new-contributor 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
63-23317
2 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR large-import new-contributor 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
63-23316
2 months 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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR new-contributor t-measure-probability 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
60-65110
1 month 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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-computability merge-conflict awaiting-author awaiting-zulip 307/5 Mathlib/Computability/NFA.lean 1 27 ['TpmKranz', 'YaelDillies', 'dupuisf', 'github-actions', 'leanprover-community-bot-assistant', 'meithecatte', 'rudynicolop'] nobody
58-40451
1 month ago
unknown
unknown
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] [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-computability merge-conflict awaiting-author awaiting-zulip 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
57-56692
1 month ago
unknown
unknown
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-computability merge-conflict awaiting-author awaiting-zulip 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
57-55782
1 month ago
unknown
unknown
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP new-contributor merge-conflict help-wanted t-analysis 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
57-8149
1 month ago
unknown
unknown
13442 dignissimus
author:dignissimus
feat: mabel tactic for multiplicative abelian groups Mabel tactic for multiplicative abelian groups (#10361) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor merge-conflict modifies-tactic-syntax awaiting-author help-wanted t-meta 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
57-7885
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-algebra new-contributor
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
57-7883
1 month ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-category-theory new-contributor 112/0 Mathlib.lean,Mathlib/CategoryTheory/Sites/CoveringFamilies.lean 2 21 ['AnthonyBordg', 'adamtopaz', 'dagurtomas', 'github-actions', 'joelriou', 'mathlib4-merge-conflict-bot'] nobody
57-7754
1 month ago
unknown
unknown
17587 kmill
author:kmill
feat: Sym2-as-Finset theory --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-data new-contributor 105/3 Mathlib/Combinatorics/SimpleGraph/Basic.lean,Mathlib/Combinatorics/SimpleGraph/Finite.lean,Mathlib/Data/Sym/Sym2.lean,Mathlib/RingTheory/Polynomial/Vieta.lean 4 11 ['FordUniver', 'YaelDillies', 'github-actions', 'kmill', 'mathlib4-merge-conflict-bot'] nobody
57-7600
1 month ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-computability new-contributor 526/0 Mathlib.lean,Mathlib/Computability/Timed/InsertionSort.lean,Mathlib/Computability/Timed/Merge.lean,Mathlib/Computability/Timed/MergeSort.lean,Mathlib/Computability/Timed/Split.lean 5 9 ['github-actions', 'mathlib4-merge-conflict-bot'] nobody
57-7598
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-computability awaiting-zulip new-contributor 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
57-7460
1 month ago
unknown
unknown
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`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra new-contributor awaiting-CI large-import merge-conflict
label:t-algebra$
169/0 Mathlib/Algebra/Free.lean 1 12 ['YaelDillies', 'github-actions', 'mathlib4-merge-conflict-bot'] nobody
57-7320
1 month ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-computability awaiting-author new-contributor 70/0 Mathlib.lean,Mathlib/Computability/PDA.lean 2 35 ['YaelDillies', 'github-actions', 'madvorak', 'mathlib4-merge-conflict-bot', 'shetzl'] nobody
57-7314
1 month ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-category-theory new-contributor 312/0 Mathlib.lean,Mathlib/CategoryTheory/Topos/Power.lean 2 3 ['github-actions', 'joelriou', 'mathlib4-merge-conflict-bot'] b-mehta
assignee:b-mehta
57-7305
1 month ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-computability awaiting-author new-contributor 383/0 Mathlib.lean,Mathlib/Computability/LeftmostDerivation.lean 2 55 ['YaelDillies', 'github-actions', 'madvorak', 'mathlib4-merge-conflict-bot', 'shetzl'] YaelDillies
assignee:YaelDillies
57-7303
1 month ago
unknown
unknown
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. merge-conflict awaiting-author t-analysis new-contributor 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
57-7292
1 month ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-combinatorics new-contributor 187/0 Mathlib.lean,Mathlib/Combinatorics/SimpleGraph/Cycle.lean 2 42 ['IvanRenison', 'github-actions', 'mathlib4-merge-conflict-bot', 'vlad902'] kmill
assignee:kmill
57-7139
1 month ago
unknown
unknown
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. merge-conflict awaiting-author t-number-theory new-contributor 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
57-6990
1 month ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR new-contributor t-measure-probability 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
57-6802
1 month ago
194-1808
194 days ago
15-66961
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR new-contributor t-measure-probability 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
57-6801
1 month ago
194-1756
194 days ago
15-65730
15 days
26300 igorkhavkine
author:igorkhavkine
feat(Analysis/Calculus/FDeriv): continuous differentiability from continuous partial derivatives on an open domain in a product space If a function `f : E × F → G` is continuously differentiable, then its partial derivatives along `E` and `F` are also continuous. The non-trivial converse implication holds when the partial derivatives are continuous on an open domain, and they can be added together to give the total derivative of `f`. See this [#mathlib4 > Partial derivatives @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Partial.20derivatives/near/520995477) and the containing thread for some discussion. The PR creates a new import (`Mathlib.Analysis.Calculus.FDeriv.Partial`), where other results about partial derivatives could go in the future. --- *this is the migration of #25304 to the PR-from-fork workflow* - [x] depends on: #25564 - [x] depends on: #26273 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP new-contributor merge-conflict awaiting-author t-analysis 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
57-6778
1 month ago
153-55168
153 days ago
44-74030
44 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. merge-conflict awaiting-author t-algebra new-contributor
label:t-algebra$
465/0 Mathlib.lean,Mathlib/Algebra/Polynomial/ZMod.lean 2 3 ['Ruben-VandeVelde', 'github-actions', 'mathlib4-merge-conflict-bot'] nobody
57-6630
1 month ago
172-50388
172 days ago
25-4678
25 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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-category-theory new-contributor 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
57-6625
1 month ago
86-59644
86 days ago
61-75483
61 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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-combinatorics new-contributor 1266/0 Mathlib.lean,Mathlib/Combinatorics/SimpleGraph/Triangle/IndependenceNumber.lean 2 10 ['Pjotr5', 'github-actions', 'grunweg', 'mathlib4-merge-conflict-bot'] nobody
57-6588
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-category-theory new-contributor 70/1 Mathlib/CategoryTheory/Category/Factorisation.lean 1 13 ['YunkaiZhang233', 'b-mehta', 'github-actions', 'mathlib4-merge-conflict-bot', 'robin-carlier'] nobody
57-6433
1 month ago
167-63996
167 days ago
0-2875
47 minutes
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-differential-geometry new-contributor 80/0 Mathlib.lean,Mathlib/Geometry/Manifold/ZeroDim.lean 2 14 ['fyqing', 'github-actions', 'grunweg', 'mathlib4-merge-conflict-bot', 'tb65536'] grunweg
assignee:grunweg
57-6431
1 month ago
166-38658
166 days ago
0-3675
1 hour
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. merge-conflict t-combinatorics new-contributor 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
57-6299
1 month ago
57-6300
57 days ago
99-48372
99 days
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 merge-conflict blocked-by-other-PR t-combinatorics new-contributor 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
57-6285
1 month ago
unknown
unknown
28871 JaafarTanoukhi
author:JaafarTanoukhi
feat(Combinatorics/Digraph): Tournaments Define orientations and tournaments. Related to #26771. Co-authored-by: Rida Hamadani --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-combinatorics new-contributor 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
57-6146
1 month ago
57-6147
57 days ago
71-35799
71 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) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-combinatorics new-contributor 476/0 Mathlib.lean,Mathlib/Combinatorics/Digraph/Maps.lean 2 2 ['github-actions', 'mathlib4-merge-conflict-bot'] awainverse
assignee:awainverse
57-5512
1 month ago
57-5513
57 days ago
54-81855
54 days
30105 slashbade
author:slashbade
feat: add `reap` as internal tactic --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict new-contributor large-import t-meta 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
57-5484
1 month ago
unknown
unknown
30121 idontgetoutmuch
author:idontgetoutmuch
Principal fiber bundle core A structure capturing what it means to be a principal fibre bundle. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-differential-geometry new-contributor 227/0 Mathlib.lean,Mathlib/Geometry/Manifold/PrincipalFiberBundle/PrincipalGBundle.lean 2 6 ['github-actions', 'grunweg', 'mathlib4-merge-conflict-bot'] hrmacbeth
assignee:hrmacbeth
57-5479
1 month ago
79-65335
79 days ago
24-28967
24 days
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR new-contributor t-measure-probability 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
57-5343
1 month ago
unknown
unknown
31102 JOSHCLUNE
author:JOSHCLUNE
Require LeanHammer Experimenting with adding LeanHammer as a mathlib dependency --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict new-contributor 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
57-4969
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-algebra new-contributor merge-conflict awaiting-author
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
57-2344
1 month ago
unknown
unknown
31590 SuccessMoses
author:SuccessMoses
chore: tag `commutatorElement_def` with `simp` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-algebra new-contributor
label:t-algebra$
1/0 Mathlib/Algebra/Group/Commutator.lean 1 2 ['github-actions', 'grunweg'] nobody
56-66619
1 month ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-algebraic-topology new-contributor 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
56-65760
1 month ago
unknown
unknown
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) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-algebra new-contributor
label:t-algebra$
91/0 Mathlib.lean,Mathlib/GroupTheory/SpecificGroups/BraidGroup/Basic.lean 2 22 ['github-actions', 'hannahfechtner', 'jcommelin', 'joelriou'] nobody
56-65607
1 month ago
unknown
unknown
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.  --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP new-contributor t-meta 34/4 Mathlib/Tactic/Simps/Basic.lean 1 11 ['FrederickPu', 'YaelDillies', 'fpvandoorn', 'github-actions', 'leanprover-community-bot-assistant'] nobody
56-65544
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-category-theory new-contributor merge-conflict awaiting-author 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
56-65517
1 month ago
unknown
unknown
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$. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-category-theory new-contributor 33/0 Mathlib/CategoryTheory/Limits/Types/Colimits.lean 1 5 ['github-actions', 'joelriou', 'leanprover-community-bot-assistant', 'robertmaxton42'] nobody
56-65400
1 month ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-data new-contributor 15/0 Mathlib/Data/Finset/Card.lean,Mathlib/Data/Set/Finite/Basic.lean 2 5 ['Ruben-VandeVelde', 'github-actions'] nobody
56-65311
1 month ago
198-2134
198 days ago
13-83428
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-analysis new-contributor 50/2 Mathlib/Analysis/Calculus/Deriv/Star.lean 1 15 ['emo916math', 'github-actions', 'j-loreaux', 'kckennylau'] j-loreaux
assignee:j-loreaux
56-65166
1 month ago
159-64914
159 days ago
31-69534
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-data new-contributor 22/0 Mathlib/Data/Rat/Lemmas.lean 1 33 ['github-actions', 'kim-em', 'mathlib-bors', 'pechersky', 'sinianluoye', 'themathqueen'] pechersky
assignee:pechersky
56-65083
1 month ago
88-2277
88 days ago
74-50277
74 days
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 --> [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP new-contributor merge-conflict awaiting-author t-combinatorics 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
56-65062
1 month ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-ring-theory new-contributor 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
56-64951
1 month ago
122-22281
122 days ago
1-40501
1 day
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 blocked-by-other-PR t-category-theory new-contributor merge-conflict awaiting-author 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
56-64863
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR t-analysis new-contributor 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
56-64801
1 month ago
unknown
unknown
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. awaiting-author t-measure-probability new-contributor 13/0 Mathlib/MeasureTheory/PiSystem.lean 1 14 ['EtienneC30', 'KiringYJ', 'dagurtomas', 'github-actions', 'ocfnash'] RemyDegenne
assignee:RemyDegenne
56-51259
1 month ago
56-51259
56 days ago
135-34213
135 days
29434 ntapiam
author:ntapiam
feat(NonAssoc/LieAdmissible): prove every ring/algebra is LieAdmissible -awaiting-author t-algebra new-contributor
label:t-algebra$
27/6 Mathlib/Algebra/NonAssoc/LieAdmissible/Defs.lean 1 2 ['github-actions', 'mathlib4-merge-conflict-bot'] nobody
54-49569
1 month ago
unknown
unknown
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] --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP blocked-by-other-PR new-contributor awaiting-author t-analysis 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
54-570
1 month ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics new-contributor 209/0 Mathlib/Combinatorics/SetFamily/Lindstrom.lean 1 2 ['github-actions', 'mathlib4-merge-conflict-bot'] b-mehta
assignee:b-mehta
53-73408
1 month ago
57-5167
57 days ago
31-45300
31 days
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology blocked-by-other-PR new-contributor 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
52-48080
1 month ago
unknown
unknown
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis new-contributor awaiting-author 64/5 Mathlib/Analysis/SpecialFunctions/Stirling.lean 1 15 ['FaffyWaffles', 'github-actions', 'j-loreaux', 'mathlib4-merge-conflict-bot', 'tb65536'] nobody
50-42744
1 month ago
50-42744
50 days ago
4-54198
4 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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data new-contributor 23/0 Mathlib/Data/EReal/Operations.lean 1 4 ['JovanGerb', 'LLaurance', 'dobronx1325', 'github-actions'] nobody
50-21050
1 month ago
50-77362
50 days ago
6-21252
6 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$. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis new-contributor awaiting-author 14/0 Mathlib/Analysis/Convolution.lean 1 3 ['github-actions', 'urkud'] nobody
48-7430
1 month ago
48-7430
48 days ago
0-81373
22 hours
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-analysis new-contributor 331/0 Mathlib/Analysis/Normed/Operator/SingularValues.lean 1 2 ['github-actions', 'nielsvoss'] nobody
47-44971
1 month ago
unknown
unknown
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 awaiting-author t-algebra new-contributor
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
43-62820
1 month ago
82-5827
82 days ago
35-25302
35 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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis new-contributor 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
43-35614
1 month ago
unknown
unknown
31898 ntapiam
author:ntapiam
feat(LinearAlgebra/TensorAlgebra): implement HopfAlgebra for TensorAlgebra implementation of the natural Hopf algebra structure on the TensorAlgebra new-contributor t-ring-theory 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 64 ['YaelDillies', 'github-actions', 'kckennylau', 'ntapiam'] nobody
40-65807
1 month ago
53-32620
53 days ago
0-30128
8 hours
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. t-combinatorics new-contributor awaiting-author merge-conflict 113/0 Mathlib.lean,Mathlib/Combinatorics/Enumerative/Polya.lean 2 8 ['IvanRenison', 'alreadydone', 'github-actions', 'mathlib4-merge-conflict-bot'] awainverse
assignee:awainverse
40-52569
1 month ago
49-9712
49 days ago
39-39956
39 days
31113 515801431
author:515801431
feat(Mathlib/Combinatorics/Enumerative/Polya.lean): Add additional theorem in `Polya.lean` --- - [ ] depends on: #30525 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics new-contributor blocked-by-other-PR merge-conflict 302/0 Mathlib.lean,Mathlib/Combinatorics/Enumerative/Polya.lean 2 4 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] b-mehta
assignee:b-mehta
40-52445
1 month ago
49-74871
49 days ago
16-74719
16 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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-data new-contributor 129/1 Mathlib.lean,Mathlib/Data/List/Commutativity.lean,Mathlib/Data/List/Defs.lean,Mathlib/Data/List/Lemmas.lean 4 38 ['MrSumato', 'github-actions', 'grunweg', 'madvorak', 'mathlib4-merge-conflict-bot', 'plp127'] grunweg
assignee:grunweg
40-48047
1 month ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics new-contributor 391/0 Mathlib.lean,Mathlib/Combinatorics/DiHypergraph/Basic.lean 2 2 ['github-actions', 'mathlib4-merge-conflict-bot'] b-mehta
assignee:b-mehta
37-75484
1 month ago
57-5527
57 days ago
57-67557
57 days
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-dynamics new-contributor awaiting-author 114/6 Mathlib/Dynamics/Transitive.lean 1 6 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'sgouezel'] sgouezel
assignee:sgouezel
37-73280
1 month ago
37-73280
37 days ago
18-34491
18 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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics new-contributor merge-conflict 375/0 Mathlib.lean,Mathlib/Combinatorics/Hypergraph/Basic.lean 2 54 ['b-mehta', 'espottesmith', 'github-actions', 'jt496', 'lauramonk', 'mathlib4-merge-conflict-bot'] b-mehta
assignee:b-mehta
36-6493
1 month ago
57-6283
57 days ago
76-50008
76 days
26479 thefundamentaltheor3m
author:thefundamentaltheor3m
feat(Analysis/Complex/CauchyIntegral): Cauchy–Goursat for Unbounded Rectangles In this PR, we prove versions of the Cauchy-Goursat theorem where the contours in question are rectangular and unbounded (ie, where the contours look like the $\bigsqcup$ symbol). I am not sure if I have formalised these in the best way, or if `Analysis.Complex.CauchyIntegral` is the best place for them (it might be prudent to reorganise the file into multiple files at some point), but I believe this is a useful result. Suggestions welcome. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-analysis sphere-packing 199/0 Mathlib/Analysis/Complex/CauchyIntegral.lean 1 3 ['github-actions', 'mathlib4-merge-conflict-bot', 'wwylele'] nobody
34-70949
1 month ago
unknown
unknown
32609 PrParadoxy
author:PrParadoxy
feat(LinearAlgebra/PiTensorProduct): Relation between nested tensor products and tensor products indexed by dependent sums Product tensors in `⨂ j : (Σ i, β i), s j.fst j.snd` can be mapped to product tensors in `⨂ i, ⨂ b : β i, s i b`. If the outer index type is finite, the two types are equivalent. This allows the definition of endomorphisms on PiTensorProducts by specifying them on disjoint subsets of the index set. Such constructions are common e.g. in quantum circuits, quantum cellular automata, and renormalization procedures. --- WIP. This PR contains two "requests for comments". Essentially: * Is a single complex-to-define linear equivalence preferable over several less complex ones, which might however be of limited interest by themselves? * Which trade-offs are appropriate to make things computable? - [ ] depends on: #32608 - [ ] depends on: #32600 - [x] depends on: #32598 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor blocked-by-other-PR 683/0 Mathlib.lean,Mathlib/Data/Sigma/Basic.lean,Mathlib/LinearAlgebra/Multilinear/Basic.lean,Mathlib/LinearAlgebra/PiTensorProduct/Nested.lean,Mathlib/LinearAlgebra/PiTensorProduct/Set.lean 5 4 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
34-32413
1 month ago
37-43788
37 days ago
0-614
10 minutes
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-measure-probability new-contributor awaiting-author merge-conflict 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 7 ['github-actions', 'jcommelin', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'zhuyizheng'] sgouezel
assignee:sgouezel
34-13548
1 month ago
49-64644
49 days ago
1-22579
1 day
32552 ksenono
author:ksenono
feat(SetTheory/Cardinal): helpers for Konig's theorem --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-set-theory new-contributor 70/0 Mathlib/SetTheory/Cardinal/Arithmetic.lean,Mathlib/SetTheory/Cardinal/Basic.lean 2 33 ['SnirBroshi', 'b-mehta', 'github-actions', 'ksenono', 'staroperator', 'vihdzp'] b-mehta
assignee:b-mehta
32-15389
1 month ago
32-36797
32 days ago
37-79310
37 days
32869 felixpernegger
author:felixpernegger
feat(RingTheory): lemmas around ```Ring.choose``` Various small lemmas around Ring.choose. In particular this should cover all statements from .Data.Nat.Choose.Basic which have a meaningful generalization to arbitrary rings. new-contributor t-ring-theory 170/0 Mathlib/RingTheory/Binomial.lean,Mathlib/RingTheory/Polynomial/Pochhammer.lean 2 1 ['github-actions'] nobody
32-1745
1 month ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-measure-probability new-contributor awaiting-author 21/0 Mathlib/Probability/Moments/Basic.lean 1 5 ['DavidLedvinka', 'github-actions'] RemyDegenne
assignee:RemyDegenne
31-65386
1 month ago
31-65386
31 days ago
21-30654
21 days
32600 PrParadoxy
author:PrParadoxy
feat(LinearAlgebra/Multilinear): composition of multilinear maps The composition of a multilinear map with a family of multilinear maps is a multilinear map indexed by a dependent sum. The result reduces to a lemma about the interaction of function application, `Sigma.curry`, and `Function.update`. This variant of `Function.apply_update` is included as `Sigma.apply_curry_update`. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor 40/0 Mathlib/Data/Sigma/Basic.lean,Mathlib/LinearAlgebra/Multilinear/Basic.lean 2 4 ['github-actions', 'goliath-klein', 'kbuzzard'] dwrensha
assignee:dwrensha
31-60260
1 month ago
unknown
unknown
31766 SuccessMoses
author:SuccessMoses
feat(Topology/EMetricSpace): continuity of arc length fixes half of #31751 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-topology awaiting-author 396/0 Mathlib.lean,Mathlib/Topology/EMetricSpace/ArcLength.lean,Mathlib/Topology/EMetricSpace/BoundedVariation.lean 3 39 ['SnirBroshi', 'SuccessMoses', 'alreadydone', 'github-actions', 'grunweg', 'j-loreaux'] nobody
30-82373
30 days ago
36-43223
36 days ago
2-76065
2 days
32555 ksenono
author:ksenono
feat(Combinatorics/SimpleGraph/Matching): maximum and maximal matchings for Konig's theorem --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics new-contributor 127/1 Mathlib/Combinatorics/SimpleGraph/DegreeSum.lean,Mathlib/Combinatorics/SimpleGraph/Matching.lean 2 8 ['SnirBroshi', 'github-actions', 'ksenono'] awainverse
assignee:awainverse
28-19910
28 days ago
28-18983
28 days ago
38-43127
38 days
32570 ksenono
author:ksenono
feat(Combinatorics/SimpleGraph): bipartite subgraphs and vertex-disjoint graphs for Konig's theorem --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics new-contributor 22/0 Mathlib/Combinatorics/SimpleGraph/Bipartite.lean,Mathlib/Combinatorics/SimpleGraph/Subgraph.lean 2 10 ['SnirBroshi', 'github-actions'] kmill
assignee:kmill
28-19450
28 days ago
28-18542
28 days ago
38-18442
38 days
32845 jonasvanderschaaf
author:jonasvanderschaaf
feat(CategoryTheory): `GrothendieckTopology.yoneda` preserves certain (co)limits We prove that if every `J`-sheaf preserves limits of shape `Kᵒᵖ`, then `J.yoneda` preserves colimits of shape `K`, and the dual statement. We specialize to the case of finite products, and deduce that the inclusion of light profinite sets in light condensed sets preserves finite coproducts From [LeanCondensed](https://github.com/dagurtomas/LeanCondensed) --- Co-authored-by: Dagur Asgeirsson [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor WIP 108/0 Mathlib.lean,Mathlib/CategoryTheory/Limits/Preserves/Shapes/Products.lean,Mathlib/CategoryTheory/Sites/PreservesLimits.lean,Mathlib/CategoryTheory/Sites/Subcanonical.lean,Mathlib/Condensed/Light/Functors.lean 5 1 ['github-actions'] nobody
27-61031
27 days ago
unknown
unknown
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) - [ ] depends on: #33061 **The next PR is here:** #31670 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology new-contributor awaiting-author blocked-by-other-PR 293/1 Mathlib.lean,Mathlib/Topology/Order/ScottTopology.lean,Mathlib/Topology/Order/ScottTopologyDCPO.lean,docs/references.bib 4 39 ['b-mehta', 'edwin1729', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'plp127'] b-mehta
assignee:b-mehta
27-43666
27 days ago
47-73851
47 days ago
5-43456
5 days
32938 0xTerencePrime
author:0xTerencePrime
feat(Order/LocallyFinite): prove DenselyOrdered and LocallyFiniteOrder are incompatible ## Summary This PR proves that a nontrivial densely ordered linear order cannot be locally finite. ## Main results * `not_locallyFiniteOrder`: A densely ordered locally finite linear order must be subsingleton. * `not_locallyFiniteOrder_of_nontrivial`: The main theorem - incompatibility of the two properties. Note: This implementation imports `Mathlib.Order.Interval.Set.Infinite` to reuse the existing `Set.Icc_infinite` theorem, ensuring standard library consistency. ## Mathematical content The key insight is that in a densely ordered type, we can always find a new element between any two distinct elements. This means any nontrivial interval contains infinitely many elements. However, `LocallyFiniteOrder` requires intervals to be finite. This contradiction implies that such a type cannot exist (unless it is trivial). ## Motivation This resolves a TODO mentioned in #7987 (Data/Finset/LocallyFinite entry). ## Verification - [x] `lake build Mathlib.Order.LocallyFinite.Basic` passes - [x] `lake exe runLinter Mathlib.Order.LocallyFinite.Basic` passes t-order new-contributor awaiting-author 28/0 Mathlib/Order/Interval/Finset/Basic.lean 1 10 ['0xTerencePrime', 'CoolRmal', 'github-actions', 'jcommelin', 'plp127'] nobody
27-2388
27 days ago
27-2428
27 days ago
2-83075
2 days
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebraic-topology blocked-by-other-PR new-contributor 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
26-62193
26 days ago
unknown
unknown
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`, a direct construction without ε-transitions. - Theorem `accepts_concat : (M1.concat M2).accepts = M1.accepts * M2.accepts`, showing the correctness of the construction. - Theorem `IsRegular.mul`, showing that regular languages are closed under concatenation. --- - [x] depends on: #31038 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-computability new-contributor maintainer-merge 104/7 Mathlib/Computability/NFA.lean 1 63 ['YaelDillies', 'ctchou', 'github-actions', 'lambda-fairy', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'rudynicolop'] YaelDillies
assignee:YaelDillies
26-39226
26 days ago
26-38270
26 days ago
45-11894
45 days
32698 farruhx
author:farruhx
feat(List): add aesop / simp annotations to selected lemmas for improved automation This PR adds `@[aesop safe]` and `@[simp]` annotations to a set of List lemmas whose proofs are routine and benefit from standardized automation. No statements or definitions are changed; only proof annotations are added. The lemmas updated in this PR are: * `or_exists_of_exists_mem_cons` * `append_subset_of_subset_of_subset` * `map_subset_iff` * `append_eq_has_append` * `append_right_injective` * `append_left_injective` * `reverse_surjective` * `reverse_bijective` * `mem_getLast?_append_of_mem_getLast?` * `mem_dropLast_of_mem_of_ne_getLast` * `idxOf_eq_length_iff` * `idxOf_append_of_mem` * `length_eraseP_add_one` The goal is to make these commonly used lemmas easier for `aesop`-based automation to resolve, while avoiding any interference with simp-normal-form lemmas or canonical rewrite rules. There are no API changes and no new theorems—only improved automation behavior. t-data new-contributor awaiting-author 18/1 Mathlib/Data/List/Basic.lean 1 8 ['artie2000', 'euprunin', 'farruhx', 'github-actions'] pechersky
assignee:pechersky
26-37157
26 days ago
26-37157
26 days ago
7-30937
7 days
32826 felixpernegger
author:felixpernegger
feat(Data/Tuple/Sort): Permutation is monotone iff its the identity Sort of permutation is its inverse + Permutation is monotone iff its the identity t-data new-contributor 19/0 Mathlib/Data/Fin/Tuple/Sort.lean 1 1 ['github-actions'] TwoFX
assignee:TwoFX
26-31272
26 days ago
30-75519
30 days ago
33-21577
33 days
29953 slashbade
author:slashbade
feat: add reap for experiment --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
26-19244
26 days ago
unknown
unknown
27817 zhuyizheng
author:zhuyizheng
feat: add IMO2025P1 Add a solution to IMO2025P1, the original problem statement from https://github.com/jsm28/IMOLean --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) IMO awaiting-author new-contributor merge-conflict 1310/0 Archive.lean,Archive/Imo/Imo2025Q1.lean 2 9 ['github-actions', 'kim-em', 'mathlib4-merge-conflict-bot', 'zhuyizheng'] dwrensha
assignee:dwrensha
25-69354
25 days ago
85-33922
85 days ago
54-69322
54 days
32910 felixpernegger
author:felixpernegger
feat(Data/Nat/Choose): two binomial coefficient sum identities This PR proves two well-known sum identities around binomial coefficients. While there are probably hundreds of such identities, these two seem to be well known enough to be in mathlib (i.e. are mentioned in the Wikipedia [article](https://en.wikipedia.org/wiki/Binomial_coefficient#math_8) about binomial coefficients). new-contributor t-data 31/0 Mathlib/Data/Nat/Choose/Sum.lean,Mathlib/Data/Nat/Choose/Vandermonde.lean 2 1 ['github-actions'] TwoFX
assignee:TwoFX
25-31242
25 days ago
30-65061
30 days ago
30-64881
30 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 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] --> [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author new-contributor large-import 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
25-29725
25 days ago
115-84846
115 days ago
2-2914
2 days
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). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology new-contributor awaiting-author 110/18 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
24-15580
24 days ago
47-62982
47 days ago
8-9680
8 days
26923 oliver-butterley
author:oliver-butterley
feat(Dynamics/BirkhoffSum): add the pointwise ergodic theorem (Birkhoff's) The Pointwise Ergodic Theorem, also known as Birkhoff's Ergodic Theorem. Co-authored-by: Lua Viana Reis - [x] depends on: #26074 - [x] depends on: #26807 - [x] depends on: #26810 - [x] depends on: #26840 - [x] depends on: #26842 - [x] depends on: #26848 - [x] depends on: #26851 - [x] depends on: #26852 - [x] depends on: #26853 - [x] depends on: #27008 - [x] depends on: #28901 Zulip: [PR thread](https://leanprover.zulipchat.com/#narrow/channel/144837-PR-reviews/topic/.2326923.20The.20pointwise.20ergodic.20theorem.20.28Birkhoff's.29/with/527835158) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-dynamics new-contributor awaiting-author 398/0 Mathlib.lean,Mathlib/Dynamics/BirkhoffSum/Pointwise.lean 2 31 ['D-Thomine', 'github-actions', 'leanprover-community-bot-assistant', 'lua-vr', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'sgouezel', 'urkud'] sgouezel
assignee:sgouezel
24-5377
24 days ago
29-49695
29 days ago
98-42878
98 days
33031 chiyunhsu
author:chiyunhsu
feat(Combinatorics/Enumerative/Partition): add combinatorial proof of Euler's partition theorem The new file EulerComb.lean contains the combinatorial proof of Euler's partition theorem. The analytic proof of the theorem and its generalization of Glaisher's Theorem has already been formalized in [Glaisher.lean](https://github.com/leanprover-community/mathlib4/blob/master/Mathlib/Combinatorics/Enumerative/Partition/Glaisher.lean). The generalization of the combinatorial proof from this file to Glaisher's Theorem is within reach. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics new-contributor 531/0 Mathlib.lean,Mathlib/Combinatorics/Enumerative/Partition/EulerComb.lean 2 5 ['chiyunhsu', 'github-actions', 'tb65536', 'vihdzp'] b-mehta
assignee:b-mehta
23-31261
23 days ago
28-3017
28 days ago
28-2837
28 days
33109 felixpernegger
author:felixpernegger
feat(Data/Nat/Choose): Binomial inversion This PR adds binomial inversion (also called binomial transform), which is a useful method for proving binomial identities. It is tricky to find direct references to binomial inversion, but for example [this](https://en.wikipedia.org/wiki/Binomial_transform#Binomial_convolution) Wikipedia article mentions it ("The formula"). The first theorem ```alternating_sum_choose_mul_of_alternating_sum_choose_mul``` could be refined (we only need the hypothesis ```h``` up to some point), but this seems to needlessly complicate it. new-contributor 107/0 Mathlib.lean,Mathlib/Data/Nat/Choose/Inversion.lean 2 4 ['felixpernegger', 'github-actions', 'wwylele'] dagurtomas
assignee:dagurtomas
23-31251
23 days ago
25-62272
25 days ago
26-4033
26 days
33218 Blackfeather007
author:Blackfeather007
feat(Algebra): Define the associated graded ring to filtered ring Define the associated graded ring to a filtered ring. --- - [ ] depends on: #33217 migrated from https://github.com/leanprover-community/mathlib4/pull/26858 t-ring-theory new-contributor blocked-by-other-PR 450/0 Mathlib.lean,Mathlib/RingTheory/FilteredAlgebra/AssociatedGraded.lean 2 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
23-15619
23 days ago
unknown
unknown
33219 Blackfeather007
author:Blackfeather007
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: #33218 migrated from #26859 t-ring-theory new-contributor blocked-by-other-PR 563/0 Mathlib.lean,Mathlib/RingTheory/FilteredAlgebra/AssociatedGraded.lean 2 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
23-15511
23 days ago
unknown
unknown
33220 Blackfeather007
author:Blackfeather007
feat(Algebra): Define associated graded module Define the associated graded module to a filtered module. --- - [ ] depends on: #33218 migrated from #26860 t-ring-theory new-contributor blocked-by-other-PR 669/0 Mathlib.lean,Mathlib/RingTheory/FilteredAlgebra/AssociatedGraded.lean 2 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
23-15427
23 days ago
unknown
unknown
33227 Blackfeather007
author:Blackfeather007
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 [suzuka@misaka-yu.com](mailto:suzuka@misaka-yu.com) Co-authored-by: Yi Yuan @yuanyi-350 [kysyy1@126.com](mailto:kysyy1@126.com) Co-authored-by: Weichen Jiao @AlbertJ-314 [albertjiao314@gmail.com](mailto:albertjiao314@gmail.com) --- - [ ] depends on: #33226 migrated from #26869 t-ring-theory new-contributor blocked-by-other-PR 728/0 Mathlib.lean,Mathlib/RingTheory/FilteredAlgebra/AssociatedGraded.lean,Mathlib/RingTheory/FilteredAlgebra/Exactness.lean,Mathlib/RingTheory/FilteredAlgebra/FilteredHom.lean 4 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
23-13099
23 days ago
23-13100
23 days ago
0-206
3 minutes
33226 Blackfeather007
author:Blackfeather007
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 [suzuka@misaka-yu.com](mailto:suzuka@misaka-yu.com) Co-authored-by: Yi Yuan @yuanyi-350 [kysyy1@126.com](mailto:kysyy1@126.com) Co-authored-by: Weichen Jiao @AlbertJ-314 [albertjiao314@gmail.com](mailto:albertjiao314@gmail.com) --- - [ ] depends on: #33222 migrated from #26868 t-ring-theory new-contributor blocked-by-other-PR 529/0 Mathlib.lean,Mathlib/RingTheory/FilteredAlgebra/AssociatedGraded.lean,Mathlib/RingTheory/FilteredAlgebra/Exactness.lean,Mathlib/RingTheory/FilteredAlgebra/FilteredHom.lean 4 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
23-13097
23 days ago
23-13098
23 days ago
0-415
6 minutes
33225 Blackfeather007
author:Blackfeather007
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: #33220 - [ ] depends on: #33223 migrated from #26867 t-ring-theory new-contributor blocked-by-other-PR 1205/0 Mathlib.lean,Mathlib/RingTheory/FilteredAlgebra/AssociatedGraded.lean,Mathlib/RingTheory/FilteredAlgebra/FilteredHom.lean 3 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
23-13096
23 days ago
unknown
unknown
33224 Blackfeather007
author:Blackfeather007
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: #33219 - [ ] depends on: #33223 migrated from #26863 t-ring-theory new-contributor blocked-by-other-PR 1055/0 Mathlib.lean,Mathlib/RingTheory/FilteredAlgebra/AssociatedGraded.lean,Mathlib/RingTheory/FilteredAlgebra/FilteredHom.lean 3 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
23-13094
23 days ago
23-13095
23 days ago
0-978
16 minutes
33223 Blackfeather007
author:Blackfeather007
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 [suzuka@misaka-yu.com](mailto:suzuka@misaka-yu.com) Co-authored-by: Yi Yuan @yuanyi-350 [kysyy1@126.com](mailto:kysyy1@126.com) Co-authored-by: Weichen Jiao @AlbertJ-314 [albertjiao314@gmail.com](mailto:albertjiao314@gmail.com) --- - [ ] depends on: #33218 - [ ] depends on: #33222 migrated from #26862 t-ring-theory new-contributor blocked-by-other-PR 824/0 Mathlib.lean,Mathlib/RingTheory/FilteredAlgebra/AssociatedGraded.lean,Mathlib/RingTheory/FilteredAlgebra/FilteredHom.lean 3 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
23-13091
23 days ago
23-13094
23 days ago
0-1162
19 minutes
33222 Blackfeather007
author:Blackfeather007
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 [suzuka@misaka-yu.com](mailto:suzuka@misaka-yu.com) Co-authored-by: Yi Yuan @yuanyi-350 [kysyy1@126.com](mailto:kysyy1@126.com) Co-authored-by: Weichen Jiao @AlbertJ-314 [albertjiao314@gmail.com](mailto:albertjiao314@gmail.com) --- - [ ] depends on: #33217 migrated from #26861 new-contributor t-ring-theory blocked-by-other-PR 368/0 Mathlib.lean,Mathlib/RingTheory/FilteredAlgebra/AssociatedGraded.lean,Mathlib/RingTheory/FilteredAlgebra/FilteredHom.lean 3 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
23-13090
23 days ago
23-13091
23 days ago
0-1375
22 minutes
33178 gw90
author:gw90
feat(Analysis/CStarAlgebra/Spectrum): Adding lemmas that the CStarAlgebra norm equals the square root of the spectral radius of star a * a Adds lemmas that the ||a||^2_A=sqrt(spectralRadius C (star a * a)). I think it would be helpful to have these lemmas available in Mathlib. It'll help with some of the other things I'm working on. Feel free to move them to a different file or rename them as you see fit. new-contributor t-analysis awaiting-author 24/0 Mathlib/Analysis/CStarAlgebra/Spectrum.lean 1 15 ['github-actions', 'gw90', 'themathqueen', 'vihdzp'] nobody
22-51358
22 days ago
24-26977
24 days ago
0-14336
3 hours
31092 FlAmmmmING
author:FlAmmmmING
feat(Algebra/Group/ForwardDiff.lean): Add theorem `sum_shift_eq_fwdDiff_iter`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra new-contributor
label:t-algebra$
17/1 Mathlib/Algebra/Group/ForwardDiff.lean 1 18 ['BeibeiX0', 'FlAmmmmING', 'Ruben-VandeVelde', 'dagurtomas', 'github-actions', 'mathlib4-merge-conflict-bot'] dagurtomas
assignee:dagurtomas
21-6634
21 days ago
21-5473
21 days ago
46-81323
46 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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory new-contributor awaiting-author 527/0 Mathlib.lean,Mathlib/CategoryTheory/Bicategory/LaxSlice.lean 2 12 ['dagurtomas', 'github-actions', 'jjtowery', 'robin-carlier'] dagurtomas
assignee:dagurtomas
19-41576
19 days ago
unknown
unknown
32546 anishrajeev
author:anishrajeev
feat(ModelTheory): Prove compactness of the type space Define the space of types and prove various topological properties of it (zero dimensional, totally separated, compact, baire). The goal is to formalize the proof of the Omitting Types Theorem - [ ] depends on: #32215 t-logic new-contributor blocked-by-other-PR 127/1 Mathlib.lean,Mathlib/ModelTheory/Topology/Types.lean,Mathlib/ModelTheory/Types.lean,Mathlib/Tactic/Linter/DirectoryDependency.lean 4 5 ['NoneMore', 'anishrajeev', 'github-actions', 'mathlib4-dependent-issues-bot'] fpvandoorn
assignee:fpvandoorn
19-12775
19 days ago
34-62807
34 days ago
3-63673
3 days
32960 dleijnse
author:dleijnse
feat(FieldTheory): adjoin pth roots For a field `k` of exponential characteristic `p` and a subset `S` of `k`, we define the extension of `k` obtained by adjoining all `p`-th roots of elements of `S`. We prove that this is a purely inseparable extension, and provide some basic API. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra new-contributor awaiting-author
label:t-algebra$
131/0 Mathlib.lean,Mathlib/FieldTheory/PurelyInseparable/AdjoinPthRoots.lean 2 13 ['artie2000', 'chrisflav', 'dleijnse', 'erdOne', 'github-actions', 'leanprover-radar'] erdOne
assignee:erdOne
18-58228
18 days ago
18-58228
18 days ago
10-11880
10 days
33163 Aaron1011
author:Aaron1011
feat: prove subgroup of (M -> Z) is finitely generated --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-ring-theory new-contributor awaiting-author 5/0 Mathlib/RingTheory/DedekindDomain/Dvr.lean 1 2 ['erdOne', 'github-actions'] alreadydone
assignee:alreadydone
18-51178
18 days ago
18-51178
18 days ago
5-78603
5 days
33217 Blackfeather007
author:Blackfeather007
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. --- migrated from https://github.com/leanprover-community/mathlib4/pull/26857 new-contributor t-ring-theory awaiting-author 144/0 Mathlib.lean,Mathlib/RingTheory/FilteredAlgebra/AssociatedGraded.lean 2 4 ['erdOne', 'github-actions'] erdOne
assignee:erdOne
18-45519
18 days ago
18-45519
18 days ago
4-55780
4 days
33280 michelsol
author:michelsol
feat(MeasureTheory/Integral/IntervalIntegral): add variant `integral_deriv_eq_sub_uIoo` of 2nd theorem of calculus. Add a continuous on uIcc, differentiable on uIoo, deriv version of the 2nd fundamental theorem of calculus. This corresponds to what is written [here](https://en.wikipedia.org/wiki/Fundamental_theorem_of_calculus#Second_part). For example it makes it easier to compute the integral : ```lean4 ∫ x : ℝ in 0..1, (√(1 - x ^ 2))⁻¹ = ∫ x : ℝ in 0..1, deriv arcsin x = arcsin 1 - arcsin 0 ``` It is not possible to use [`interval_deriv_eq_sub`](https://leanprover-community.github.io/mathlib4_docs/Mathlib/MeasureTheory/Integral/IntervalIntegral/FundThmCalculus.html#intervalIntegral.integral_deriv_eq_sub) which requires differentiability on all of [0,1], as `arcsin` isn't differentiable at 1. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-measure-probability new-contributor 14/0 Mathlib/MeasureTheory/Integral/IntervalIntegral/FundThmCalculus.lean 1 1 ['github-actions'] EtienneC30
assignee:EtienneC30
17-31243
17 days ago
20-55888
20 days ago
20-55708
20 days
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 45 ['BoltonBailey', 'IlPreteRosso', 'TwoFX', 'github-actions', 'kckennylau', 'mathlib4-merge-conflict-bot', 'rudynicolop'] TwoFX
assignee:TwoFX
17-20161
17 days ago
26-38102
26 days ago
90-59512
90 days
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`. t-combinatorics new-contributor 76/0 Mathlib.lean,Mathlib/Combinatorics/Enumerative/RecLatticePath.lean 2 3 ['github-actions', 'mathlib4-merge-conflict-bot'] awainverse
assignee:awainverse
16-83520
16 days ago
16-82697
16 days ago
36-28736
36 days
33021 farmanb
author:farmanb
feat(RingTheory/IdealFilter): add ideal filters and Gabriel filters This PR introduces ideal filters on a ring and the notion of a Gabriel filter. Main additions: * `IdealFilter A`: filters on the lattice of ideals of a ring `A` * `IsUniform`: the uniformity (T1–T3) condition * `gabrielComposition` and notation `•` * `IsGabriel`: Gabriel filters (axiom T4) * A characterization `IsGabriel ↔ IsUniform ∧ F • F = F` This is preparatory infrastructure for future work relating Gabriel filters to Giraud subcategories. This development is motivated by Theorem 10.2 in Bo Stenström, *Rings and Modules of Quotients*, which identifies equivalence classes of Giraud subcategories with linear (Gabriel) topologies on a ring. The present PR provides the ring-theoretic filter infrastructure needed for that result. --- - [ ] depends on: #33390 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-ring-theory new-contributor blocked-by-other-PR 283/0 Mathlib.lean,Mathlib/RingTheory/Ideal/Colon.lean,Mathlib/RingTheory/IdealFilter/Basic.lean,docs/references.bib 4 21 ['erdOne', 'farmanb', 'github-actions', 'mathlib4-dependent-issues-bot'] mattrobball
assignee:mattrobball
15-63489
15 days ago
15-63490
15 days ago
11-73862
11 days
33133 0xTerencePrime
author:0xTerencePrime
feat(Algebra/Group/Center): add Decidable (IsMulCentral a) instance This PR adds a `Decidable` instance for `IsMulCentral a`. ### Summary The structure `IsMulCentral` was missing a `Decidable` instance. This PR provides the instance by leveraging `isMulCentral_iff`, enabling decidability for both multiplicative and additive (via `to_additive`) structures. ### Verification - `lake build Mathlib.Algebra.Group.Center` passed. - `lake exe runLinter Mathlib.Algebra.Group.Center` passed. t-algebra new-contributor awaiting-author
label:t-algebra$
7/0 Mathlib/Algebra/Group/Center.lean 1 3 ['github-actions', 'robin-carlier'] ocfnash
assignee:ocfnash
12-79369
12 days ago
12-79369
12 days ago
12-58151
12 days
33276 NicolaBernini
author:NicolaBernini
feat: Rename List.reverse_perm to List.reverse_perm_self and List.reverse_perm' to List.reverse_perm_iff --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor awaiting-author 17/15 Mathlib/Algebra/BigOperators/Group/List/Basic.lean,Mathlib/Data/Finset/Dedup.lean,Mathlib/Data/List/Basic.lean,Mathlib/Data/List/Defs.lean,Mathlib/Data/List/Perm/Lattice.lean,Mathlib/Data/List/Permutation.lean,Mathlib/Data/Multiset/Defs.lean,Mathlib/NumberTheory/Divisors.lean 8 4 ['Ruben-VandeVelde', 'github-actions'] kim-em
assignee:kim-em
12-68503
12 days ago
16-78697
16 days ago
3-79472
3 days
33481 NoneMore
author:NoneMore
feat(ModelTheory/Encoding): add `Countable` instances for (bounded) formulas in countable languages Prepare for the OTT proof. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-logic new-contributor 27/0 Mathlib/ModelTheory/Encoding.lean 1 1 ['github-actions'] nobody
12-15015
12 days ago
12-14079
12 days ago
12-81800
12 days
33520 NoneMore
author:NoneMore
feat(ModelTheory/ElementarySubstructures): add a variant of Tarski-Vaught test taking sets as input There should exist an `ElementarySubstructure.copy` such that we can directly bundle the set itself instaed of its closure as an elementary substructure. The other direction depends on #33458. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-logic new-contributor 63/0 Mathlib/ModelTheory/ElementarySubstructures.lean 1 1 ['github-actions'] nobody
11-68454
11 days ago
11-79857
11 days ago
11-79677
11 days
33463 khwilson
author:khwilson
feat(Mathlib/Analysis/Polynomial/MahlerMeasure): Mahler Measure for other rings Define `mahlerMeasure'` which allows you specify a norm preserving map `v` from any `NormedRing A` (or more general) to `ℂ`. Also provide wrappers around the main `mahlerMeasure` lemmas that are used for estimation. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor 96/2 Mathlib/Analysis/Polynomial/MahlerMeasure.lean,Mathlib/NumberTheory/MahlerMeasure.lean 2 16 ['github-actions', 'khwilson', 'plp127', 'vlad902'] nobody
11-64316
11 days ago
unknown
unknown
32608 PrParadoxy
author:PrParadoxy
feat(LinearAlgebra/PiTensorProduct): API for PiTensorProducts indexed by sets This PR addresses a TODO item in LinearAlgebra/PiTensorProduct.lean: * API for the various ways ι can be split into subsets; connect this with the binary tensor product -- specifically by describing tensors of type ⨂ (i : S), M i, for S : Set ι. Our primary motivation is to formalise the notion of "restricted tensor products". This will be the content of a follow-up PR. Beyond that, the Set API is natural in contexts where the index type has an independent interpretation. An example is quantum physics, where ι ranges over distinguishable degrees of freedom, and where its is common practice to annotate objects by the set of indices they are defined on. --- Stub file with preliminary definition of the restricted tensor product as a direct limit of tensors indexed by finite subsets of an index type: https://github.com/PrParadoxy/mathlib4/blob/restricted-stub/Mathlib/LinearAlgebra/PiTensorProduct/Restricted.lean --- - [x] depends on: #32598 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor awaiting-zulip 300/2 Mathlib.lean,Mathlib/LinearAlgebra/PiTensorProduct.lean,Mathlib/LinearAlgebra/PiTensorProduct/Set.lean 3 28 ['PrParadoxy', 'dagurtomas', 'eric-wieser', 'github-actions', 'goliath-klein', 'leanprover-radar', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] dagurtomas
assignee:dagurtomas
11-59342
11 days ago
23-59045
23 days ago
10-63624
10 days
33502 MrQubo
author:MrQubo
fix(Tactic/ProxyType): Pass params explicitly in proxy_equiv% implementation Fix [#mathlib4 > `deriving Fintype` with Prop](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/.60deriving.20Fintype.60.20with.20Prop/with/566118621) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-meta WIP 12/2 Mathlib/Tactic/ProxyType.lean,MathlibTest/DeriveFintype.lean 2 7 ['MrQubo', 'github-actions', 'kmill'] kmill
assignee:kmill
11-46293
11 days ago
11-46294
11 days ago
0-57325
15 hours
22657 Xmask19
author:Xmask19
feat: a graph is maximally acyclic iff it is a tree --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-combinatorics new-contributor 86/0 Mathlib/Combinatorics/SimpleGraph/Acyclic.lean 1 8 ['Rida-Hamadani', 'SnirBroshi', 'b-mehta', 'github-actions', 'grunweg', 'mathlib4-merge-conflict-bot'] b-mehta
assignee:b-mehta
11-39386
11 days ago
unknown
unknown
33247 sun123zxy
author:sun123zxy
feat(Mathlib/RingTheory/Ideal/Cotangent): dimension of cotangent spaces It is shown that the span rank of the maximal ideal of a local ring equals the dimension of the cotangent space if the maximal ideal is finitely generated. To avoid unnecessary imports, the original `Mathlib/RingTheory/Nakayama` is now moved to `Mathlib/RingTheory/Nakayama/Basic`. --- - [ ] depends on: #33359 - [ ] depends on: #33361 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) file-removed new-contributor t-ring-theory blocked-by-other-PR WIP merge-conflict 314/20 Mathlib.lean,Mathlib/Algebra/Module/SpanRank.lean,Mathlib/RingTheory/Ideal/Cotangent.lean,Mathlib/RingTheory/Ideal/KrullsHeightTheorem.lean,Mathlib/RingTheory/LocalRing/Module.lean,Mathlib/RingTheory/LocalRing/Quotient.lean,Mathlib/RingTheory/Nakayama/Basic.lean,Mathlib/RingTheory/Nakayama/SpanRank.lean,Mathlib/RingTheory/Regular/RegularSequence.lean,Mathlib/RingTheory/Support.lean 10 11 ['erdOne', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'sun123zxy'] nobody
10-78801
10 days ago
18-45837
18 days ago
3-69477
3 days
32978 archiebrowne
author:archiebrowne
feat(NumberTheory/ModularForms/Basic): Provide definition of the products of finitely many modular forms `finprod_equal_weights`: the product of n modular forms of weight k is a modular form of weight n * k `inprod_add_weights`: the product of n modular forms of different weights has weight the sum of the weights new-contributor t-number-theory awaiting-author 97/18 Mathlib/NumberTheory/ModularForms/Basic.lean,Mathlib/NumberTheory/ModularForms/NormTrace.lean,Mathlib/NumberTheory/ModularForms/SlashActions.lean,Mathlib/NumberTheory/ModularForms/SlashInvariantForms.lean,Mathlib/Order/Filter/ZeroAndBoundedAtFilter.lean 5 19 ['archiebrowne', 'github-actions', 'loefflerd', 'wwylele'] loefflerd
assignee:loefflerd
9-74211
9 days ago
27-1679
27 days ago
2-44108
2 days
33601 nielstron
author:nielstron
feat(Computability/ContextFreeGrammar): Concatenation of CFGs is CFG --- - [ ] depends on: #33599 - [ ] depends on: #33592 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-computability new-contributor blocked-by-other-PR 946/0 Mathlib/Computability/ContextFreeGrammar.lean 1 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
9-71660
9 days ago
unknown
unknown
33599 nielstron
author:nielstron
feat(Computability/ContextFreeGrammar): closure under union --- This PR picks up https://github.com/leanprover-community/mathlib4/pull/13514 and resolves the outstanding errors. - [ ] depends on #33592 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-computability new-contributor 506/0 Mathlib/Computability/ContextFreeGrammar.lean 1 1 ['github-actions'] nobody
9-65133
9 days ago
9-71029
9 days ago
9-70849
9 days
17176 arulandu
author:arulandu
feat: integrals and integrability with .re Lemmas for swapping order of .re and integration/integrability. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author new-contributor t-measure-probability please-adopt 49/0 Mathlib/MeasureTheory/Function/L1Space.lean,Mathlib/MeasureTheory/Integral/IntegrableOn.lean,Mathlib/MeasureTheory/Integral/IntervalIntegral.lean,Mathlib/MeasureTheory/Integral/SetIntegral.lean 4 32 ['EtienneC30', 'arulandu', 'github-actions', 'loefflerd'] nobody
9-49291
9 days ago
unknown
unknown
32918 michelsol
author:michelsol
feat: define `supEdist` and `supDist` Create a new file Topology.MetricSpace.SupDistance and define the supremal distance in (extended) metric spaces. The defined `supEdist` and `supDist` will have similar theory to the already existing `infEdist` and `infDist`. The motivation is to be able to define the radius of a minimal bounding sphere as the infimum of the supDist later. [zulip discussion here](https://leanprover.zulipchat.com/#narrow/channel/116395-maths/topic/Formalizing.20Jung's.20theorem.20and.20minimal.20bounding.20spheres) t-topology new-contributor merge-conflict 75/0 Mathlib.lean,Mathlib/Topology/MetricSpace/SupDistance.lean 2 2 ['github-actions', 'mathlib4-merge-conflict-bot'] RemyDegenne
assignee:RemyDegenne
9-48692
9 days ago
9-48694
9 days ago
21-957
21 days
33281 michelsol
author:michelsol
feat(Analysis/SpecialFunctions/Integrals): integral of 1/sqrt(1-x^2) and its integrability. Add the integral of the derivative of arcsin and its integrability. --- - [ ] depends on: #33280 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor blocked-by-other-PR merge-conflict 59/0 Mathlib/Analysis/SpecialFunctions/Integrability/Basic.lean,Mathlib/Analysis/SpecialFunctions/Integrals/Basic.lean,Mathlib/MeasureTheory/Integral/IntervalIntegral/FundThmCalculus.lean 3 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
9-35221
9 days ago
20-54035
20 days ago
0-811
13 minutes
33458 NoneMore
author:NoneMore
feat(ModelTheory): add lifting for embeddings to languages with constants Prepare for a generalized Tarski-Vaught test with a set as input instead of a substructure. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-logic new-contributor 46/0 Mathlib/ModelTheory/ElementaryMaps.lean,Mathlib/ModelTheory/LanguageMap.lean 2 1 ['github-actions'] fpvandoorn
assignee:fpvandoorn
9-31254
9 days ago
13-1906
13 days ago
13-1726
13 days
33061 edwin1729
author:edwin1729
refactor: generalise compact from CompleteLattice to PartialOrder `IsCompactElement` assumes a `CompleteLattice` structure on the type for which it is defined. But a `PartialOrder` will suffice and this is the textbook definition of compact https://en.wikipedia.org/wiki/Compact_element. Also it is currently defined in a non-standard way. The standard definition uses directed sets. Changing this has indeed simplified most proofs by removing an `rw` into this more standard form. --- Note to reviewers: moving `IsCompactElement` out of the `CompleteLattice` namespace caused the loss of being able to use dot notation [here](https://github.com/leanprover-community/mathlib4/pull/33061/changes#diff-2e06453359871b8a74315294d1f7825b7b5aa1221c69b4e058893b2c9418230fR498) and [here](https://github.com/leanprover-community/mathlib4/pull/33061/changes#diff-1d4a166e29849096ebe0e5d25bd4dc5f97db1d3b8caf1703177034160e77a310R350). Would like help fixing that [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor awaiting-author 84/63 Mathlib/Algebra/Lie/Submodule.lean,Mathlib/LinearAlgebra/Span/Basic.lean,Mathlib/Order/BooleanGenerators.lean,Mathlib/Order/CompactlyGenerated/Basic.lean,Mathlib/Order/CompactlyGenerated/Intervals.lean,Mathlib/RingTheory/Finiteness/Basic.lean,Mathlib/RingTheory/Ideal/Span.lean,Mathlib/RingTheory/Spectrum/Prime/Topology.lean,Mathlib/Topology/Sets/Opens.lean 9 11 ['b-mehta', 'edwin1729', 'github-actions', 'plp127'] nobody
8-84556
8 days ago
26-61186
26 days ago
0-70180
19 hours
33257 NickAdfor
author:NickAdfor
feat(Combinatorics/SimpleGraph/Bipartite): Odd Cycle Theorem (A Solution to TODO) Prove bipartite iff all cycles are even This PR formalizes the classical graph theory theorem: a graph is bipartite if and only if all its cycles have even length. Co-authored-by: Nick Adfor Co-authored-by: Yue Sun Co-authored-by: Aristotle AI --- ## Main results - `SimpleGraph.bipartite_iff_all_cycles_even` : the main equivalence theorem ## Key supporting lemmas - `SimpleGraph.even_length_iff_same_color` : parity lemma for 2-colorings - `SimpleGraph.even_length_iff_even_bypass_length` : bypass length parity - `SimpleGraph.even_cycle_length_of_path` : cycle construction lemma - `SimpleGraph.bypass_eq_nil_of_closed` : closed path properties ## Proof outline 1. For bipartite graphs: use the 2-coloring to show that in a 2-coloring, a walk has even length iff its endpoints have the same color. 2. For cycles (start = end), this forces even length. 3. For the converse: if all cycles are even, construct a 2-coloring using the `two_colorable_iff_forall_loop_even` characterization. 4. Show this coloring is valid using bypass operations and path properties. ## Technical notes - Uses `SimpleGraph.Walk` for path/cycle representation - Handles both `IsPath` and `IsCycle` predicates - Uses bypass operations (`takeUntil`, `dropUntil`, `bypass`) to analyze walks - Requires `DecidableEq V` for some lemmas - Uses classical logic for case analysis ## Reviewer notes - The proof uses induction on walks and case analysis on colorings - Some lemmas (like `even_length_iff_same_color`) could be extracted to more general locations - All theorems are in the `SimpleGraph` namespace - The `bipartite_iff_all_cycles_even` theorem provides the complete characterization t-combinatorics new-contributor awaiting-author 141/5 Mathlib/Combinatorics/SimpleGraph/Bipartite.lean,Mathlib/Combinatorics/SimpleGraph/ConcreteColorings.lean 2 42 ['IvanRenison', 'NickAdfor', 'Rida-Hamadani', 'SnirBroshi', 'github-actions', 'kmill', 'mitchell-horner', 'vihdzp'] nobody
8-70778
8 days ago
unknown
unknown
33032 ksenono
author:ksenono
feat(Combinatorics/SimpleGraph): Konig’s theorem on bipartite graphs --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics new-contributor blocked-by-other-PR merge-conflict 983/2 Mathlib.lean,Mathlib/Combinatorics/SimpleGraph/Basic.lean,Mathlib/Combinatorics/SimpleGraph/Bipartite.lean,Mathlib/Combinatorics/SimpleGraph/Clique.lean,Mathlib/Combinatorics/SimpleGraph/DegreeSum.lean,Mathlib/Combinatorics/SimpleGraph/Konig/Auxillary.lean,Mathlib/Combinatorics/SimpleGraph/Konig/Konig.lean,Mathlib/Combinatorics/SimpleGraph/Konig/KonigFin.lean,Mathlib/Combinatorics/SimpleGraph/Maps.lean,Mathlib/Combinatorics/SimpleGraph/Matching.lean,Mathlib/Combinatorics/SimpleGraph/Subgraph.lean,Mathlib/Combinatorics/SimpleGraph/VertexCover.lean,Mathlib/SetTheory/Cardinal/Arithmetic.lean,Mathlib/SetTheory/Cardinal/Basic.lean 14 8 ['SnirBroshi', 'github-actions', 'ksenono', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'vlad902'] nobody
8-69554
8 days ago
unknown
unknown
33592 nielstron
author:nielstron
feat(Computability/ContextFreeGrammar): mapping between two types of nonterminal symbols --- This PR picks up https://github.com/leanprover-community/mathlib4/pull/15895 and resolves the failing lemma by redefining Good symbols. I checked that https://github.com/leanprover-community/mathlib4/pull/13514 builds correctly when based on this build. PR for that is #33599 This is my first contribution please let me know of any changes I should outline. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-computability new-contributor 162/0 Mathlib/Computability/ContextFreeGrammar.lean 1 1 ['github-actions', 'madvorak'] nobody
8-66767
8 days ago
9-76141
9 days ago
9-75961
9 days
32742 LTolDe
author:LTolDe
feat(MeasureTheory/Constructions/Polish/Basic): add class SuslinSpace add new class `SuslinSpace` for a topological space that is an analytic set in itself This will be useful to prove the **Effros Theorem**, see [zulip thread](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Effros.20Theorem/with/558712441). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor awaiting-zulip 4/0 Mathlib/MeasureTheory/Constructions/Polish/Basic.lean 1 9 ['ADedecker', 'LTolDe', 'dupuisf', 'github-actions', 'jcommelin'] PatrickMassot
assignee:PatrickMassot
8-65927
8 days ago
8-66080
8 days ago
11-6345
11 days
33050 mkaratarakis
author:mkaratarakis
feat: lemmas for the analytic part of the proof of the Gelfond–Schneider theorem Lemmas missing for the formalisation of the proof of the Gelfond–Schneider theorem --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-number-theory new-contributor awaiting-author 221/0 Mathlib.lean,Mathlib/Analysis/Analytic/Basic.lean,Mathlib/Analysis/Analytic/Order.lean,Mathlib/Analysis/Complex/CauchyIntegral.lean,Mathlib/NumberTheory/Transcendental/AnalyticPart.lean 5 105 ['SnirBroshi', 'github-actions', 'j-loreaux', 'mkaratarakis', 'riccardobrasca', 'vihdzp'] riccardobrasca
assignee:riccardobrasca
8-37118
8 days ago
8-51222
8 days ago
5-6442
5 days
33389 khwilson
author:khwilson
feat(Mathlib/Analysis/SpecialFunctions/Log/Base): More log asymptotics A common utility in proving asymptotics is `logb b =O[⊤] log` and `(log ∘ (c * ·)) =O[atTop] log` and related lemmas `logb`. This PR fills these in for future use. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis new-contributor awaiting-author 28/2 Mathlib/Analysis/SpecialFunctions/Log/Base.lean 1 16 ['github-actions', 'j-loreaux', 'khwilson', 'vlad902'] j-loreaux
assignee:j-loreaux
8-20542
8 days ago
8-66362
8 days ago
7-54803
7 days
32583 MJ141592
author:MJ141592
refactor(SimpleGraph): change bridges not to require the edge to be present Remove the requirement for edges to exist in definition of isBridge, and then change the related lemmas to adjust for this, by renaming, fixing the statements and fixing the proofs, including in Acyclic. Closes #31690. t-combinatorics new-contributor awaiting-author 60/47 Mathlib/Combinatorics/SimpleGraph/Acyclic.lean,Mathlib/Combinatorics/SimpleGraph/Connectivity/Connected.lean 2 15 ['MJ141592', 'SnirBroshi', 'YaelDillies', 'github-actions', 'mathlib4-merge-conflict-bot'] nobody
7-73278
7 days ago
37-51741
37 days ago
0-20559
5 hours
28708 sjh227
author:sjh227
feat(LinearAlgebra): define row- and column-stochastic matrices This PR defines row- and column-stochastic matrices, and relates them to doubly stochastic matrices (which are already in mathlib). --- t-data new-contributor 255/6 Mathlib.lean,Mathlib/Algebra/Group/Submonoid/Defs.lean,Mathlib/Analysis/Convex/DoublyStochasticMatrix.lean,Mathlib/LinearAlgebra/Matrix/Stochastic.lean 4 29 ['dupuisf', 'github-actions', 'j-loreaux', 'mathlib4-merge-conflict-bot', 'sjh227'] pechersky
assignee:pechersky
7-31265
7 days ago
10-43516
10 days ago
10-54841
10 days
33330 michael-novak-math
author:michael-novak-math
feat: add arc-length reparametrization of parametrized curves add new definitions of arc-length reparametrization and its corresponding parameter transformation and a theorem establishing the desired properties. t-analysis new-contributor merge-conflict 311/0 Mathlib.lean,Mathlib/Analysis/Calculus/ArcLengthReparametrization.lean,Mathlib/MeasureTheory/Integral/IntervalIntegral/FundThmCalculus.lean,docs/references.bib,lake-manifest.json 5 53 ['SnirBroshi', 'github-actions', 'grunweg', 'j-loreaux', 'mathlib4-merge-conflict-bot', 'michael-novak-math'] j-loreaux
assignee:j-loreaux
7-30246
7 days ago
7-30247
7 days ago
6-57754
6 days

PRs not into the master branch

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
13158 erdOne
author:erdOne
refactor(RingTheory/OreLocalization/Module): remove `LocalizedModule.mk`. --- - [x] depends on: #13151 - [ ] depends on: #13156 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra blocked-by-other-PR
label:t-algebra$
49/48 Mathlib/RingTheory/OreLocalization/Basic.lean,Mathlib/RingTheory/OreLocalization/Module.lean 2 2 ['leanprover-community-mathlib4-bot', 'urkud'] nobody
3-19692
3 days ago
unknown
unknown

PRs with an 'approved' review

Number Author Title Description Labels +/- Modified files (first 100) 📝 💬 All users who commented or reviewed Assignee(s) Approval(s) Updated Last status change total time in review
12608 eric-wieser
author:eric-wieser
feat: allow `nsmul` / `zsmul` to be omitted again, with a warning --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-algebra t-meta
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 1
533-5308
1 year ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-algebra
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 1
533-5305
1 year ago
unknown
unknown
9146 laughinggas
author:laughinggas
feat(Data/ZMod/Defs): Topological structure on `ZMod` Added a discrete topology structure to `ZMod n` for all `n` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra awaiting-author t-topology
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 1
533-5305
1 year ago
unknown
unknown
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') ``` [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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 1
533-5304
1 year ago
unknown
unknown
6403 astrainfinita
author:astrainfinita
chore: change instance priorities of `Ordered*` hierarchy --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-order merge-conflict slow-typeclass-synthesis 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 1
533-5303
1 year ago
unknown
unknown
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`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-data new-contributor 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 1
513-69005
1 year ago
unknown
unknown
15448 urkud
author:urkud
chore(*): deprecate `Option.elim'` Use `Option.elim` instead. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author tech debt 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 1
513-58058
1 year ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-topology 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 2
464-18440
1 year ago
unknown
unknown
13514 madvorak
author:madvorak
feat(Computability/ContextFreeGrammar): closure under union - [ ] depends on: #15895 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-computability blocked-by-other-PR 448/4 Mathlib/Computability/ContextFreeGrammar.lean 1 50 ['Rida-Hamadani', 'YaelDillies', 'github-actions', 'leanprover-community-mathlib4-bot', 'madvorak'] nobody 1
438-84862
1 year ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-topology t-order 34/14 Mathlib/Topology/Constructions.lean,Mathlib/Topology/Order/LowerUpperTopology.lean 2 13 ['Ruben-VandeVelde', 'TwoFX', 'github-actions', 'jcommelin', 'mans0954', 'mathlib-bors', 'riccardobrasca'] nobody 2
426-4510
1 year ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-algebra new-contributor
label:t-algebra$
78/0 Mathlib/Algebra/Group/Defs.lean 1 13 ['github-actions', 'hannahfechtner', 'jcommelin', 'kbuzzard', 'kim-em', 'trivial1711'] nobody 1
360-977
11 months ago
unknown
unknown
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? --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-meta 12/1 Mathlib/Tactic/Linarith/Preprocessing.lean 1 3 ['Vierkantor', 'harahu', 'kim-em', 'mo271'] nobody 1
349-69397
11 months ago
unknown
unknown
19189 YnirPaz
author:YnirPaz
feat(SetTheory/Ordinal/Arithmetic): order isomorphism between omega and the natural numbers --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-set-theory 44/0 Mathlib/Order/SuccPred/Limit.lean,Mathlib/SetTheory/Ordinal/Arithmetic.lean 2 21 ['YaelDillies', 'YnirPaz', 'github-actions', 'vihdzp'] nobody 1
300-24380
9 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict delegated 8/0 lakefile.lean 1 20 ['YaelDillies', 'adomani', 'eric-wieser', 'github-actions', 'grunweg', 'mathlib-bors'] nobody 1
285-69241
9 months ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
1
279-85759
9 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) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) This is started from the mathport output on https://github.com/leanprover-community/mathlib/pull/19244 merge-conflict t-analysis awaiting-zulip 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 1
265-32503
8 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-data 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 1
253-42364
8 months ago
unknown
unknown
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) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra t-analysis awaiting-CI
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 1
251-69478
8 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-logic 62/0 Mathlib/ModelTheory/Substructures.lean 1 19 ['GabinKolly', 'YaelDillies', 'fpvandoorn', 'github-actions', 'grunweg'] nobody 1
250-60438
8 months ago
unknown
unknown
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-linter large-import merge-conflict awaiting-author delegated 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 1
243-63263
7 months ago
unknown
unknown
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.) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-linter 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
1
233-76593
7 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-differential-geometry 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
1
194-20751
6 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-meta 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
1
154-36826
5 months ago
unknown
unknown
26078 kckennylau
author:kckennylau
feat(AlgebraicGeometry): add x, y, px, py for points on elliptic curves --- Split from #25218. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-algebraic-geometry 44/0 Mathlib/AlgebraicGeometry/EllipticCurve/Affine/Point.lean 1 12 ['MichaelStollBayreuth', 'Multramate', 'acmepjz', 'dagurtomas', 'github-actions', 'kckennylau'] dagurtomas
assignee:dagurtomas
1
146-66442
4 months ago
146-66442
146 days ago
64-10273
64 days
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-data new-contributor 24/26 Mathlib/Data/TypeVec.lean 1 7 ['Equilibris', 'alexkeizer', 'github-actions', 'mathlib4-merge-conflict-bot'] nobody 1
145-36748
4 months ago
145-36749
145 days ago
13-47613
13 days
26462 PSchwahn
author:PSchwahn
feat(LinearAlgebra/Projection): add results about inverse of `Submodule.prodEquivOfIsCompl` Add two theorems `Submodule.prodEquivOfIsCompl_symm_apply` and `Submodule.prodEquivOfIsCompl_symm_add`, which are API for `Submodule.prodEquivOfIsCompl`. We believe these theorems are useful; for example, we have used their statements in a [classification formalization project](https://github.com/LieLean/LowDimSolvClassification). Co-authored by: - [Viviana del Barco](https://github.com/vdelbarc) - [Gustavo Infanti](https://github.com/GuQOliveira) - [Exequiel Rivas](https://github.com/erivas) --- I am not sure whether the `prodEquivOfIsCompl_symm_apply` theorem should be tagged with `@[simp]`; this might lead to confluence issues. Opinions are welcome! [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-algebra new-contributor
label:t-algebra$
10/0 Mathlib/LinearAlgebra/Projection.lean 1 7 ['PSchwahn', 'github-actions', 'joelriou', 'kckennylau'] joelriou
assignee:joelriou
1
128-35429
4 months ago
128-66532
128 days ago
73-38219
73 days
27937 madvorak
author:madvorak
feat(Logic/Basic): `congr_heq₂` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-logic 6/0 Mathlib/Logic/Basic.lean 1 8 ['YaelDillies', 'fpvandoorn', 'github-actions', 'madvorak', 'vihdzp'] fpvandoorn
assignee:fpvandoorn
1
119-85768
3 months ago
146-153
145 days ago
17-59565
17 days
21950 erdOne
author:erdOne
feat(NumberTheory/Padics): the completion of `ℚ` at a finite place is `ℚ_[p]` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-number-theory 253/1 Mathlib.lean,Mathlib/Algebra/GroupWithZero/WithZero.lean,Mathlib/NumberTheory/Padics/HeightOneSpectrum.lean,Mathlib/NumberTheory/Padics/PadicNumbers.lean,Mathlib/Topology/Algebra/Valued/WithVal.lean,Mathlib/Topology/Algebra/WithZeroMulInt.lean,Mathlib/Topology/Algebra/WithZeroTopology.lean 7 33 ['Ruben-VandeVelde', 'erdOne', 'faenuccio', 'github-actions', 'leanprover-community-bot-assistant', 'pechersky', 'smmercuri', 'xroblot'] nobody 1
110-69282
3 months ago
unknown
unknown
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 awaiting-author t-data 360/0 MathlibTest/Junk.lean 1 17 ['SnirBroshi', 'Timeroot', 'bryangingechen', 'github-actions', 'leanprover-community-bot-assistant', 'madvorak', 'pechersky', 'vihdzp'] pechersky
assignee:pechersky
2
107-26609
3 months ago
107-26609
107 days ago
33-15711
33 days
27302 tristan-f-r
author:tristan-f-r
feat(Fintype/Quotient): finLiftOn₂ The combination of [`Quotient.finLiftOn`](https://leanprover-community.github.io/mathlib4_docs/Mathlib/Data/Fintype/Quotient.html#Quotient.finLiftOn) and [`liftOn₂`](https://leanprover-community.github.io/mathlib4_docs/Init/Core.html#Quotient.liftOn%E2%82%82). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-data 19/0 Mathlib/Data/Fintype/Quotient.lean 1 12 ['github-actions', 'kckennylau', 'pechersky', 'tristan-f-r', 'vihdzp'] pechersky
assignee:pechersky
2
91-17369
2 months ago
91-17369
91 days ago
5-78194
5 days
28925 grunweg
author:grunweg
chore: remove `linear_combination'` tactic When `linear_combination` was refactored in #15899, the old code was kept as the `linear_combination'` tactic, for easier migration. The consensus of the zulip discussion ([#mathlib4 > Narrowing the scope of `linear_combination` @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Narrowing.20the.20scope.20of.20.60linear_combination.60/near/470237816)) was to wait, and "revisit this once people have experienced the various tactics in practice". One year later, the old tactic has almost no uses: it is unused in mathlib; [searching on github](https://github.com/search?q=linear_combination%27%20path%3A*.lean&type=code) yields 37 hits --- all of which are in various forks of mathlib. Thus, removing this tactic seems appropriate. --- Do not merge before the zulip discussion has concluded! [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict file-removed awaiting-zulip 0/564 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/LinearCombination'.lean,Mathlib/Tactic/Linter/UnusedTactic.lean,MathlibTest/linear_combination'.lean 5 4 ['euprunin', 'github-actions', 'grunweg', 'mathlib4-merge-conflict-bot'] nobody 1
91-12445
2 months ago
unknown
unknown
28737 astrainfinita
author:astrainfinita
refactor: deprecate `MulEquivClass` This PR continues the work from #18806. Original PR: https://github.com/leanprover-community/mathlib4/pull/18806 merge-conflict awaiting-author t-algebra
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
1
79-2927
2 months ago
142-49500
142 days ago
2-23111
2 days
27180 ADedecker
author:ADedecker
feat: quotient of a monoid with zero by a multiplicative congruence --- My motivation is getting a more conceptual construction of [ValuativeRel.ValueGroupWithZero](https://leanprover-community.github.io/mathlib4_docs/Mathlib/RingTheory/Valuation/ValuativeRel.html#ValuativeRel.ValueGroupWithZero), but I think this is of independent interest. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra delegated
label:t-algebra$
141/26 Mathlib.lean,Mathlib/Data/Quot.lean,Mathlib/Data/Setoid/Basic.lean,Mathlib/GroupTheory/Congruence/Defs.lean,Mathlib/GroupTheory/Congruence/GroupWithZero.lean 5 32 ['ADedecker', 'eric-wieser', 'github-actions', 'mathlib-bors', 'mathlib4-merge-conflict-bot', 'ocfnash'] ocfnash
assignee:ocfnash
1
75-72583
2 months ago
155-1718
155 days ago
27-80433
27 days
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. merge-conflict awaiting-author tech debt t-analysis 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 10 ['ADedecker', 'b-mehta', 'github-actions', 'j-loreaux', 'mathlib4-merge-conflict-bot', 'mcdoll', 'plp127'] nobody 1
61-68332
2 months ago
64-55704
64 days ago
2-74132
2 days
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-bench t-linter large-import merge-conflict awaiting-author t-meta 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 71 ['Command-Master', 'Vierkantor', 'github-actions', 'grunweg', 'kmill', 'leanprover-bot', 'mathlib4-merge-conflict-bot', 'thorimur', 'urkud'] nobody 1
59-38623
1 month ago
unknown
unknown
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) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-analysis 404/0 Mathlib.lean,Mathlib/Analysis/Calculus/Gradient/Lemmas.lean 2 31 ['chenyili0818', 'github-actions', 'jcommelin', 'mathlib4-merge-conflict-bot', 'sgouezel', 'winstonyin'] nobody 1
57-8021
1 month ago
unknown
unknown
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) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-linter 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 1
57-7890
1 month ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-computability 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 1
57-7456
1 month ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-category-theory 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 1
57-7446
1 month ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-computability awaiting-author new-contributor 70/0 Mathlib.lean,Mathlib/Computability/PDA.lean 2 35 ['YaelDillies', 'github-actions', 'madvorak', 'mathlib4-merge-conflict-bot', 'shetzl'] nobody 1
57-7314
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-data 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
1
57-7288
1 month ago
unknown
unknown
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`) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-data 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
1
57-6604
1 month ago
57-6605
57 days ago
133-15886
133 days
27163 pechersky
author:pechersky
feat(Topology/ValuativeRel): of and to basis of compatible valuations --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) - [x] depends on: #30262 t-number-theory t-algebra merge-conflict awaiting-author t-topology
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
1
57-6587
1 month ago
58-38378
58 days ago
62-47306
62 days
27534 PierreQuinton
author:PierreQuinton
feat: a typeclass for `sSup`/`sInf` to be lawful Adds lawful infima and suprema type classes. A preorder with lawful suprema: whenever a set has a least upper bound, `sSup` returns a least upper bound for that set. A preorder with lawful infima: whenever a set has a greatest lower bound, `sInf` returns a greastest lower bound for that set. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-order 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
1
57-6441
1 month ago
57-6442
57 days ago
114-33795
114 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` ] --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-topology t-order large-import 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
1
57-6292
1 month ago
61-60970
61 days ago
93-38369
93 days
28871 JaafarTanoukhi
author:JaafarTanoukhi
feat(Combinatorics/Digraph): Tournaments Define orientations and tournaments. Related to #26771. Co-authored-by: Rida Hamadani --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-combinatorics new-contributor 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
1
57-6146
1 month ago
57-6147
57 days ago
71-35799
71 days
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) please-adopt merge-conflict t-topology awaiting-zulip 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 1
56-65726
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-algebra
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
1
56-65138
1 month ago
148-62159
148 days ago
7-8492
7 days
26975 Whysoserioushah
author:Whysoserioushah
feat: a norm_num extension for complex numbers co-authored-by : @thefundamentaltheor3m, @hrmacbeth --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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 1
51-42488
1 month ago
70-44565
70 days ago
111-3153
111 days
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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 2
50-17088
1 month ago
68-79400
68 days ago
9-65641
9 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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-data merge-conflict 44/22 Mathlib/Data/Int/GCD.lean 1 6 ['astrainfinita', 'b-mehta', 'eric-wieser', 'github-actions', 'mathlib4-merge-conflict-bot', 'nomeata', 'urkud'] nobody 1
48-80946
1 month 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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author merge-conflict 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 1
44-35474
1 month ago
51-84726
51 days ago
6-67021
6 days
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order awaiting-author merge-conflict 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
1
41-14509
1 month ago
44-75503
44 days ago
24-12813
24 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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-meta merge-conflict 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 7 ['JovanGerb', 'fpvandoorn', 'github-actions', 'mathlib4-merge-conflict-bot', 'thorimur'] thorimur
assignee:thorimur
2
40-63076
1 month ago
54-60581
54 days ago
7-68317
7 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]`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-order merge-conflict 8/2 Mathlib/Order/SuccPred/Basic.lean 1 4 ['YaelDillies', 'github-actions', 'mathlib4-merge-conflict-bot', 'plp127', 'vihdzp'] bryangingechen
assignee:bryangingechen
1
40-27675
1 month ago
117-43383
117 days ago
44-7812
44 days
30666 erdOne
author:erdOne
feat(NumberTheory): every number field has a ramified prime --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-number-theory awaiting-author t-algebra merge-conflict
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 23 ['erdOne', 'github-actions', 'jcommelin', 'mathlib4-merge-conflict-bot', 'tb65536', 'xroblot'] jcommelin
assignee:jcommelin
1
34-12624
1 month ago
67-27521
67 days ago
13-60954
13 days
32552 ksenono
author:ksenono
feat(SetTheory/Cardinal): helpers for Konig's theorem --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-set-theory new-contributor 70/0 Mathlib/SetTheory/Cardinal/Arithmetic.lean,Mathlib/SetTheory/Cardinal/Basic.lean 2 33 ['SnirBroshi', 'b-mehta', 'github-actions', 'ksenono', 'staroperator', 'vihdzp'] b-mehta
assignee:b-mehta
1
32-15389
1 month ago
32-36797
32 days ago
37-79310
37 days
31766 SuccessMoses
author:SuccessMoses
feat(Topology/EMetricSpace): continuity of arc length fixes half of #31751 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-topology awaiting-author 396/0 Mathlib.lean,Mathlib/Topology/EMetricSpace/ArcLength.lean,Mathlib/Topology/EMetricSpace/BoundedVariation.lean 3 39 ['SnirBroshi', 'SuccessMoses', 'alreadydone', 'github-actions', 'grunweg', 'j-loreaux'] nobody 1
30-82373
30 days ago
36-43223
36 days ago
2-76065
2 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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) I found this being not-simp frustrating when talking about submodules over a valuation subring. merge-conflict t-algebra
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 26 ['artie2000', 'eric-wieser', 'github-actions', 'j-loreaux', 'kckennylau', 'leanprover-bot', 'leanprover-radar', 'linesthatinterlace', 'mathlib4-merge-conflict-bot', 'pechersky'] joelriou
assignee:joelriou
1
30-38311
30 days ago
51-74260
51 days ago
60-49993
60 days
26608 vihdzp
author:vihdzp
feat(SetTheory/Cardinal/Aleph): `o.card ≤ ℵ_ o` and variants --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-set-theory 24/0 Mathlib/SetTheory/Cardinal/Aleph.lean 1 4 ['artie2000', 'github-actions', 'kckennylau', 'leanprover-community-bot-assistant', 'vihdzp'] alreadydone
assignee:alreadydone
2
29-66800
29 days ago
29-74567
29 days ago
59-56107
59 days
32828 Hagb
author:Hagb
feat(Algebra/Order/Group/Defs): add `IsOrderedAddMonoid.toIsOrderedCancelAddMonoid'` It is similar to `IsOrderedAddMonoid.toIsOrderedCancelAddMonoid`, while with different hypotheses. The conclusion `IsOrderedCancelMonoid α` on `IsOrderedAddMonoid.toIsOrderedCancelAddMonoid` still holds when the hypothesis `CommGroup α` is weakened to `CancelCommMonoid α` while `PartialOrder α` is strengthened to `LinearOrder α`. --- [`IsOrderedAddMonoid.toIsOrderedCancelAddMonoid`](https://leanprover-community.github.io/mathlib4_docs/find/?pattern=IsOrderedAddMonoid.toIsOrderedCancelAddMonoid#doc) and `IsOrderedAddMonoid.toIsOrderedCancelAddMonoid'`: https://github.com/leanprover-community/mathlib4/blob/97f78b1a4311fed1844b94f1c069219a48a098e1/Mathlib/Algebra/Order/Group/Defs.lean#L52-L62 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
4/0 Mathlib/Algebra/Order/Group/Defs.lean 1 1 ['artie2000', 'github-actions'] eric-wieser
assignee:eric-wieser
1
29-31268
29 days ago
33-7652
33 days ago
0-9883
2 hours
32570 ksenono
author:ksenono
feat(Combinatorics/SimpleGraph): bipartite subgraphs and vertex-disjoint graphs for Konig's theorem --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics new-contributor 22/0 Mathlib/Combinatorics/SimpleGraph/Bipartite.lean,Mathlib/Combinatorics/SimpleGraph/Subgraph.lean 2 10 ['SnirBroshi', 'github-actions'] kmill
assignee:kmill
1
28-19450
28 days ago
28-18542
28 days ago
38-18442
38 days
32679 YaelDillies
author:YaelDillies
chore(Data/Sym2): improve defeq of `diagSet` #30559 introduced a regression on the defeqs in the `SimpleGraph` API. This PR fixes it. From LeanCamCombi --- I personally think this new `diagSet` definition is unnecessary: `{e | e.IsDiag}` is not much longer to write than `Sym2.diagSet` and more transparent, but whatever. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data 52/41 Mathlib/Combinatorics/SimpleGraph/Basic.lean,Mathlib/Combinatorics/SimpleGraph/DeleteEdges.lean,Mathlib/Combinatorics/SimpleGraph/Operations.lean,Mathlib/Data/Sym/Card.lean,Mathlib/Data/Sym/Sym2.lean 5 9 ['SnirBroshi', 'YaelDillies', 'b-mehta', 'github-actions', 'mathlib4-merge-conflict-bot', 'vihdzp'] pechersky
assignee:pechersky
1
27-42874
27 days ago
27-41048
27 days ago
33-80987
33 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`, a direct construction without ε-transitions. - Theorem `accepts_concat : (M1.concat M2).accepts = M1.accepts * M2.accepts`, showing the correctness of the construction. - Theorem `IsRegular.mul`, showing that regular languages are closed under concatenation. --- - [x] depends on: #31038 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-computability new-contributor maintainer-merge 104/7 Mathlib/Computability/NFA.lean 1 63 ['YaelDillies', 'ctchou', 'github-actions', 'lambda-fairy', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'rudynicolop'] YaelDillies
assignee:YaelDillies
2
26-39226
26 days ago
26-38270
26 days ago
45-11894
45 days
32739 Rida-Hamadani
author:Rida-Hamadani
chore(SimpleGraph): golf and improve style of `Subwalks.lean` maintaining the sub-walks file after the walk split, golfing some proofs --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics 11/18 Mathlib/Combinatorics/SimpleGraph/Walks/Subwalks.lean 1 1 ['github-actions', 'vlad902'] awainverse
assignee:awainverse
1
25-31245
25 days ago
34-180
34 days ago
34-0
34 days
32889 artie2000
author:artie2000
feat(Algebra): forgetful lemmas for `map` and `comap` on substructures * Standardise the form of forgetful lemmas for `map` and `comap` (ie, `(co)map_toSubfoo`) * Add missing lemmas of this form * Mark all such lemmas as `simp` --- - [ ] depends on: #21031 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra awaiting-author blocked-by-other-PR merge-conflict
label:t-algebra$
72/17 Mathlib/Algebra/Algebra/NonUnitalSubalgebra.lean,Mathlib/Algebra/Algebra/Subalgebra/Basic.lean,Mathlib/Algebra/Group/Subgroup/Map.lean,Mathlib/Algebra/Module/Submodule/Map.lean,Mathlib/Algebra/Ring/Subsemiring/Basic.lean,Mathlib/Algebra/Star/Subalgebra.lean 6 30 ['YaelDillies', 'artie2000', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'vihdzp'] nobody 1
18-70684
18 days ago
28-46919
28 days ago
2-51242
2 days
33381 urkud
author:urkud
feat: add a version of the Schwarz lemma Add a version of the Schwarz lemma that is midway between the original lemma and Pick's version. Use it to show that a function that is separately holomorphic on a polydisc and is bounded on this polydisc must be continuous on it. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) - [ ] depends on: #33368 - [x] depends on: #33362 t-analysis blocked-by-other-PR merge-conflict 475/91 Mathlib.lean,Mathlib/Analysis/Complex/Schwarz.lean,Mathlib/Analysis/Complex/UnitDisc/Basic.lean,Mathlib/Analysis/Complex/UnitDisc/Schwarz.lean,Mathlib/Analysis/Complex/UnitDisc/Shift.lean 5 22 ['girving', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'urkud'] nobody 1
15-14717
15 days ago
16-69597
16 days ago
0-38
38 seconds
32654 YaelDillies
author:YaelDillies
feat(Combinatorics): a clique has size at most the chromatic number There already exists a version of this lemma for cliques given by a set, but it's impractical to provide an explicit clique on an explicit graph as a set, rather than an indexed family, especially because computing the size of the set would then involve proving that it is the range of an injective function, even though being a clique already implies being injective! Application: google-deepmind/formal-conjectures#1369 Also rename `coloringOfIsEmpty` and `colorable_of_isEmpty` to leverage anonymous dot notation, and make more arguments implicit. From FormalConjectures --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics 51/40 Mathlib/Combinatorics/SimpleGraph/Basic.lean,Mathlib/Combinatorics/SimpleGraph/Coloring.lean 2 20 ['SnirBroshi', 'YaelDillies', 'github-actions'] b-mehta
assignee:b-mehta
1
11-83106
11 days ago
11-82290
11 days ago
36-56332
36 days
32886 alreadydone
author:alreadydone
refactor(Algebra/Order): change `MulArchimedeanClass.subgroup` to `FiniteArchimedeanClass.subgroup` This gets rid of a junk value without much modification the main HahnEmbedding application. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-order
label:t-algebra$
298/157 Mathlib/Algebra/Order/Archimedean/Class.lean,Mathlib/Algebra/Order/Module/Archimedean.lean,Mathlib/Algebra/Order/Module/HahnEmbedding.lean 3 7 ['alreadydone', 'github-actions', 'vihdzp', 'wwylele'] Vierkantor
assignee:Vierkantor
1
10-43661
10 days ago
10-42788
10 days ago
31-22910
31 days
32991 artie2000
author:artie2000
chore(Algebra/Algebra): remove `Algebra.cast` coercion See discussion at https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Algebra.2Ecast/with/564501144 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict
label:t-algebra$
32/125 Mathlib/Algebra/Algebra/Basic.lean,Mathlib/Algebra/Algebra/Defs.lean,Mathlib/Algebra/Algebra/Field.lean,Mathlib/Algebra/Algebra/Subalgebra/Lattice.lean,Mathlib/Algebra/BigOperators/Expect.lean,Mathlib/Analysis/Normed/Algebra/Ultra.lean,Mathlib/FieldTheory/Differential/Liouville.lean,Mathlib/LinearAlgebra/Ray.lean,Mathlib/RingTheory/Localization/FractionRing.lean 9 11 ['Vierkantor', 'artie2000', 'github-actions', 'mathlib4-merge-conflict-bot', 'plp127', 'vihdzp'] Vierkantor
assignee:Vierkantor
1
9-58766
9 days ago
unknown
unknown
17176 arulandu
author:arulandu
feat: integrals and integrability with .re Lemmas for swapping order of .re and integration/integrability. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author new-contributor t-measure-probability please-adopt 49/0 Mathlib/MeasureTheory/Function/L1Space.lean,Mathlib/MeasureTheory/Integral/IntegrableOn.lean,Mathlib/MeasureTheory/Integral/IntervalIntegral.lean,Mathlib/MeasureTheory/Integral/SetIntegral.lean 4 32 ['EtienneC30', 'arulandu', 'github-actions', 'loefflerd'] nobody 1
9-49291
9 days ago
unknown
unknown
33592 nielstron
author:nielstron
feat(Computability/ContextFreeGrammar): mapping between two types of nonterminal symbols --- This PR picks up https://github.com/leanprover-community/mathlib4/pull/15895 and resolves the failing lemma by redefining Good symbols. I checked that https://github.com/leanprover-community/mathlib4/pull/13514 builds correctly when based on this build. PR for that is #33599 This is my first contribution please let me know of any changes I should outline. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-computability new-contributor 162/0 Mathlib/Computability/ContextFreeGrammar.lean 1 1 ['github-actions', 'madvorak'] nobody 1
8-66767
8 days ago
9-76141
9 days ago
9-75961
9 days
32165 yuanyi-350
author:yuanyi-350
feat(Real/Trigonometric): Add `sum_cos_arith_progression` and prepare for Dirichlet kernel --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis awaiting-author merge-conflict 68/0 Mathlib.lean,Mathlib/Analysis/Fourier/DirichletKernel.lean 2 8 ['BoltonBailey', 'github-actions', 'mathlib4-merge-conflict-bot', 'urkud', 'yuanyi-350'] fpvandoorn
assignee:fpvandoorn
1
8-37584
8 days ago
45-24366
45 days ago
3-70866
3 days
33192 linesthatinterlace
author:linesthatinterlace
refactor(Data/List/Induction): improve definition of `reverseRecOn` This PR improves the definition of `List.reverseRecOn`. --- This improved approach aims to give identical behavior but give a somewhat nicer proof of `List.reverseRecOn_concat`. I do not believe it is a regression in terms of performance. The approach is inspired by `biDirectionalRec`, for which I have also tweaked the definitions and proofs, albeit in a much more minor way. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data 32/27 Mathlib/Data/List/Induction.lean 1 6 ['github-actions', 'linesthatinterlace', 'vihdzp'] pechersky
assignee:pechersky
1
7-65445
7 days ago
7-64535
7 days ago
23-63368
23 days
33033 kim-em
author:kim-em
feat(Tactic/Choose): add type annotation support This PR adds support for type annotations in the `choose` tactic, similar to how `intro` supports them. This allows writing: ```lean choose (n : ℕ) (hn : n > 0) using h ``` instead of just `choose n hn using h`. The type annotation is checked against the actual type from the existential, and an error is raised if they don't match. This is useful for pedagogical purposes and for catching mistakes early. Requested on Zulip: https://leanprover.zulipchat.com/#narrow/channel/187764-Lean-for-teaching/topic/adding.20type.20annotation.20to.20.60choose.60/near/564323626 🤖 Prepared with Claude Code t-meta 170/22 Mathlib/Tactic/Choose.lean,MathlibTest/choose.lean 2 20 ['AlexKontorovich', 'eric-wieser', 'fpvandoorn', 'github-actions', 'kim-em'] joneugster
assignee:joneugster
1
7-15073
7 days ago
7-14215
7 days ago
26-38966
26 days
32744 NoneMore
author:NoneMore
feat(ModelTheory/Definablity): add `DefinableFun` definition and lemmas This PR adds two basic shapes of definable sets and `DefinableFun` definition with relevant lemmas. The main result is `Set.Definable.preimage_of_map` asserting that the preimage of a definable set under a definable map is definable. There are also some tool lemmas derived by the preimage lemma. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-logic 147/0 Mathlib/ModelTheory/Definability.lean 1 59 ['NoneMore', 'github-actions', 'mathlib4-merge-conflict-bot', 'staroperator'] fpvandoorn
assignee:fpvandoorn
1
6-10500
6 days ago
6-8979
6 days ago
33-37831
33 days
33403 xroblot
author:xroblot
feat(GroupTheory/FiniteAbelian): prove that the restriction map is surjective Let `G` be a finite commutative group and let `H` be a subgroup. If `M` is a commutative monoid such that `G →* Mˣ` and `H →* Mˣ` are both finite (this is the case for example if `M` is a commutative domain), then any homomorphism `H →* Mˣ` can be extended to an homomorphism `G →* Mˣ`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-group-theory 90/13 Mathlib/Algebra/Group/Submonoid/Operations.lean,Mathlib/GroupTheory/Exponent.lean,Mathlib/GroupTheory/FiniteAbelian/Duality.lean,Mathlib/GroupTheory/QuotientGroup/Basic.lean,Mathlib/NumberTheory/MulChar/Duality.lean,Mathlib/RingTheory/RootsOfUnity/Basic.lean 6 7 ['Ruben-VandeVelde', 'github-actions', 'xroblot'] urkud
assignee:urkud
1
5-69500
5 days ago
unknown
unknown
30640 SnirBroshi
author:SnirBroshi
feat(Combinatorics/SimpleGraph/Acyclic): acyclic and bridge theorems --- - [x] depends on: #30542 - [x] depends on: #30570 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics 76/82 Mathlib/Combinatorics/SimpleGraph/Acyclic.lean,Mathlib/Combinatorics/SimpleGraph/Connectivity/Connected.lean 2 7 ['SnirBroshi', 'b-mehta', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] b-mehta
assignee:b-mehta
1
5-46365
5 days ago
5-42599
5 days ago
36-13136
36 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`. delegated t-meta merge-conflict 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 19 ['adomani', 'b-mehta', 'eric-wieser', 'github-actions', 'grunweg', 'kim-em', 'mathlib-bors', 'mathlib4-merge-conflict-bot'] nobody 1
5-41569
5 days ago
unknown
unknown
32401 ADedecker
author:ADedecker
feat: monotonicity of D^n(U) in n and in U as CLMs --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-analysis delegated 170/3 Mathlib/Analysis/Distribution/ContDiffMapSupportedIn.lean,Mathlib/Analysis/Distribution/TestFunction.lean 2 19 ['ADedecker', 'faenuccio', 'github-actions', 'j-loreaux', 'mathlib-bors', 'mathlib4-merge-conflict-bot'] nobody 1
5-39657
5 days ago
14-44282
14 days ago
16-51391
16 days
33493 michelsol
author:michelsol
feat(RingTheory/Polynomial): An explicit formula for the Chebyshev polynomials of the first kind Adds the following explicit formula on the Chebyshev polynomial of the first kind of order n. ${ T_{n}(x)\ =\ \sum \limits _{k=0}^{\lfloor {\frac {n}{2}}\rfloor } {\binom {n}{2k}} \left(\ X^{2}-1\ \right)^{k}\ X^{n-2k}}$ This explicit formula can be found [here](https://en.wikipedia.org/wiki/Chebyshev_polynomials#Explicit_expressions). There is a proof using complex numbers but it only works if the ring R = ℂ. The proof here is by induction and works in a commutative ring R. Mathlib seems to extend the definition of Chebyshev polynomials for $n \in \mathbb{Z}$ but this would make the formula more cumbersome with `n.natAbs` in place of `n`'s, so I expressed it on `n : ℕ` directly. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-ring-theory new-contributor 51/1 Mathlib/RingTheory/Polynomial/Chebyshev.lean 1 8 ['YuvalFilmus', 'erdOne', 'github-actions', 'metakunt', 'michelsol'] erdOne
assignee:erdOne
1
4-67693
4 days ago
10-53211
10 days ago
11-43702
11 days
33604 xgenereux
author:xgenereux
feat(ValuationSubring): eq_top_iff + qol changes Given a `A : ValuationSubring K`, this PR adds the lemma `eq_top_iff : A = ⊤ ↔ ¬ A.valuation.IsNontrivial`. I have also made some small quality of life changes: 1. Added other forms of the basic rewrite lemmas with `Valuation.IsEquiv`: - `eq_zero` - `one_le_iff_one_le` - ~~`neq_one_iff_neq_one`~~ - `one_lt_iff_one_lt` - removed : `ne_zero` 2. Reorganized section following the `IsEquiv` namespace block in Valuation.Basic 3. Added lemmas `(h : v.IsEquiv v') : v.IsNontrivial ↔ v'.IsNontrivial` - `isNontrivial_of_isEquiv` - `isNontrivial_iff_isEquiv_isNontrivial` 4. Added simp tags 5. Added simp lemmas - `isNontrivial_valuationSubring_valuation_iff` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-ring-theory 69/38 Mathlib/NumberTheory/Padics/ValuativeRel.lean,Mathlib/RingTheory/Valuation/Basic.lean,Mathlib/RingTheory/Valuation/ValuationSubring.lean,Mathlib/RingTheory/Valuation/ValuativeRel/Basic.lean,Mathlib/Topology/Algebra/Valued/WithVal.lean 5 22 ['erdOne', 'github-actions', 'mathlib4-merge-conflict-bot', 'vihdzp', 'xgenereux'] nobody 1
4-58196
4 days ago
4-64352
4 days ago
4-55008
4 days
33612 xgenereux
author:xgenereux
feat(ValuationSubring): fieldTop Given a field `K`, the top element of `ValuationSubring K` is `K`, so top is also a field. Note: I fear this would be a bad instance so I have marked this as an abbrev for now. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-ring-theory 4/0 Mathlib/RingTheory/Valuation/ValuationSubring.lean 1 8 ['erdOne', 'github-actions', 'vihdzp', 'xgenereux'] mattrobball
assignee:mattrobball
1
4-57377
4 days ago
4-56442
4 days ago
9-46555
9 days
25905 mans0954
author:mans0954
feat(RingTheory/Polynomial/SmallDegreeVieta): polynomial versions of results in Algebra.QuadraticDiscriminant This PR continues the work from #25605. Original PR: https://github.com/leanprover-community/mathlib4/pull/25605 merge-conflict t-ring-theory please-adopt 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
1
4-38184
4 days ago
130-66563
130 days ago
81-61193
81 days
26614 Rida-Hamadani
author:Rida-Hamadani
feat(SimpleGraph): add more API for `take`/`drop` 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`, alongside a similar lemma for dropping vertices. --- - [x] depends on: #26655 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics 58/0 Mathlib/Combinatorics/SimpleGraph/Walks/Operations.lean,Mathlib/Combinatorics/SimpleGraph/Walks/Subwalks.lean 2 20 ['Rida-Hamadani', 'b-mehta', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] kmill
assignee:kmill
1
4-31244
4 days ago
23-25219
23 days ago
28-18879
28 days
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'` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-zulip t-logic 78/72 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,Mathlib/RingTheory/Congruence/Hom.lean 8 9 ['SnirBroshi', 'github-actions', 'mathlib4-merge-conflict-bot', 'thorimur', 'vihdzp'] thorimur
assignee:thorimur
1
4-25106
4 days ago
84-31824
84 days ago
8-45935
8 days
33254 SnirBroshi
author:SnirBroshi
feat(Data/Nat/Lattice): `¬BddAbove s → sSup s = 0` --- Note that it can also be proven `by simp [h]` after the `ConditionallyCompleteLinearOrderBot` instance below it. The theorem name matches the same theorems for other types: `Int.csSup_of_not_bdd_above`, `Real.sSup_of_not_bddAbove`, `NNReal.sSup_of_not_bddAbove`. Also renamed related `Int` theorems to conform to the naming conventions. [Zulip](https://leanprover.zulipchat.com/#narrow/channel/217875-Is-there-code-for-X.3F/topic/.60.C2.ACBddAbove.20s.20.E2.86.92.20sSup.20s.20.3D.200.60/with/565275221) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data 15/4 Mathlib/Data/Int/ConditionallyCompleteOrder.lean,Mathlib/Data/Nat/Lattice.lean 2 3 ['SnirBroshi', 'artie2000', 'github-actions', 'vihdzp'] nobody 2
3-53715
3 days ago
21-50061
21 days ago
21-69497
21 days
32971 Paul-Lez
author:Paul-Lez
feat(Data/Finsupp/Pointwise): generalise pointwise scalar multiplication of finsupps This PR continues the work from #24050. Original PR: https://github.com/leanprover-community/mathlib4/pull/24050 t-data 7/4 Mathlib/Data/Finsupp/Pointwise.lean 1 3 ['Paul-Lez', 'artie2000', 'github-actions'] pechersky
assignee:pechersky
1
3-52676
3 days ago
29-59037
29 days ago
29-58857
29 days
33760 JovanGerb
author:JovanGerb
feat(Order/Bounds/Basic): use `to_dual` - part 1 This PR uses `to_dual` in the first half of `Order/Bounds/Basic`, and in `Order/Bounds/Defs`, and also tags `Iio`/`Ioi` and `Iic`/`Ici`. This dualization went quite smoothly. The lemma `HasSubset.Subset.iscofinalfor` has been renamed to use correct capitalization (so that the name can be translated automatically), and has been deprecated. A new definition defined in this PR is `IsCoinitial` as a dual to `IsCofinal`, because `IsCoinitialFor` already existed as a dual to `IsCofinalFor`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-order 127/282 Mathlib/Order/Bounds/Basic.lean,Mathlib/Order/Bounds/Defs.lean,Mathlib/Order/Interval/Set/Defs.lean,Mathlib/Tactic/Translate/ToDual.lean 4 4 ['JovanGerb', 'github-actions', 'vihdzp'] Vierkantor
assignee:Vierkantor
1
3-31247
3 days ago
4-19277
4 days ago
4-19097
4 days
33697 artie2000
author:artie2000
feat(FieldTheory): real closed field * Define real closed fields * Prove some very basic properties --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
117/0 Mathlib.lean,Mathlib/FieldTheory/IsRealClosed/Basic.lean 2 40 ['artie2000', 'github-actions', 'vihdzp'] dagurtomas
assignee:dagurtomas
1
3-23588
3 days ago
3-51404
3 days ago
7-79671
7 days
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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 12 ['YaelDillies', 'adomani', 'github-actions', 'grunweg', 'jcommelin', 'urkud'] nobody 1
3-19599
3 days ago
unknown
unknown
32974 jano-wol
author:jano-wol
feat: golf eq_top_of_invtSubmodule_ne_bot --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) delegated t-algebra
label:t-algebra$
111/161 Mathlib/Algebra/Lie/Weights/IsSimple.lean,Mathlib/Algebra/Lie/Weights/Killing.lean,Mathlib/LinearAlgebra/RootSystem/Irreducible.lean 3 10 ['github-actions', 'jano-wol', 'mathlib-bors', 'mathlib4-merge-conflict-bot', 'ocfnash'] ocfnash
assignee:ocfnash
1
2-76577
2 days ago
2-76577
2 days ago
3-59216
3 days
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra delegated
label:t-algebra$
18/9 Mathlib/Algebra/Group/Units/Hom.lean,Mathlib/AlgebraicGeometry/Scheme.lean,Mathlib/Geometry/RingedSpace/LocallyRingedSpace.lean,Mathlib/Geometry/RingedSpace/OpenImmersion.lean,Mathlib/RingTheory/LocalRing/ResidueField/Basic.lean 5 14 ['adomani', 'alreadydone', 'erdOne', 'eric-wieser', 'github-actions', 'jcommelin', 'leanprover-community-bot-assistant', 'mathlib-bors', 'mathlib4-merge-conflict-bot', 'vihdzp'] mattrobball
assignee:mattrobball
1
2-53729
2 days ago
58-2152
58 days ago
14-54827
14 days
32880 0xTerencePrime
author:0xTerencePrime
feat(Analysis/Asymptotics): define subpolynomial growth ## Main definitions * `Asymptotics.IsSubpolynomial l f g`: A function `f` has subpolynomial growth with respect to `g` along filter `l` if `f = O(1 + ‖g‖^k)` for some natural `k`. ## Main results * `IsSubpolynomial.const`: Constant functions have subpolynomial growth * `IsSubpolynomial.id`: Identity has subpolynomial growth * `IsSubpolynomial.add`: Closure under addition * `IsSubpolynomial.neg`: Closure under negation * `IsSubpolynomial.sub`: Closure under subtraction * `IsSubpolynomial.mul`: Closure under multiplication * `IsSubpolynomial.pow`: Closure under powers * `isSubpolynomial_iff_one_add`: Equivalence with `(1 + ‖g‖)^k` formulation * `IsSubpolynomial.uniform`: Uniform bounds for finite families ## Implementation notes The definition uses `1 + ‖g‖^k` rather than `(1 + ‖g‖)^k` as the primary form, with the equivalence established in `isSubpolynomial_iff_one_add`. Four private auxiliary lemmas handle the key inequalities needed for closure proofs. Closes #32658 awaiting-author t-analysis new-contributor 185/0 Mathlib.lean,Mathlib/Analysis/Asymptotics/Subpolynomial.lean 2 28 ['0xTerencePrime', 'ADedecker', 'github-actions', 'j-loreaux'] ADedecker
assignee:ADedecker
1
2-52365
2 days ago
3-33823
3 days ago
22-12319
22 days
33504 ldct
author:ldct
feat: Add lemmas for DihedralGroup.fintypeHelper Using `fin_cases` to reason about `DihedralGroup` elements exposes the internal `fintypeHelper` instances, which has no exported API ``` example (g : DihedralGroup 3) : (g^6 = 1) := by fin_cases g <;> dsimp -- 6 goals case «0» ⊢ DihedralGroup.fintypeHelper✝ (Sum.inl 0) ^ 6 = 1 ... ``` this PR adds simp lemma that convert them to constructors, which do have API ``` 6 goals case «0» ⊢ 1 ^ 6 = 1 case «1» ⊢ DihedralGroup.r 1 ^ 6 = 1 case «2» ⊢ DihedralGroup.r 2 ^ 6 = 1 ``` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-group-theory 8/0 Mathlib/GroupTheory/SpecificGroups/Dihedral.lean 1 1 ['github-actions', 'tb65536'] nobody 1
2-12814
2 days ago
12-16151
12 days ago
12-15971
12 days
33355 0xTerencePrime
author:0xTerencePrime
feat(Combinatorics/SimpleGraph/Connectivity): define vertex connectivity This PR introduces the foundations of vertex connectivity for simple graphs, providing a counterpart to the edge connectivity theory in #32870. ### Main definitions - `SimpleGraph.IsVertexReachable`: vertices remain reachable after removing strictly fewer than `k` other vertices. - `SimpleGraph.IsVertexConnected`: a graph is `k`-vertex-connected if its order is strictly greater than `k` and any two distinct vertices are `k`-vertex-reachable. Includes basic characterizations for $k=0$ and $k=1$, along with monotonicity lemmas (`anti` and `mono`). new-contributor t-combinatorics 154/0 Mathlib.lean,Mathlib/Combinatorics/SimpleGraph/Connectivity/VertexConnectivity.lean,Mathlib/Combinatorics/SimpleGraph/IsolateVerts.lean 3 105 ['0xTerencePrime', 'SnirBroshi', 'YaelDillies', 'github-actions', 'vihdzp'] nobody 1
1-84586
1 day ago
2-52899
2 days ago
16-77184
16 days
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). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict file-removed awaiting-author t-algebra
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 11 ['Ruben-VandeVelde', 'YaelDillies', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-merge-conflict-bot', 'riccardobrasca'] riccardobrasca
assignee:riccardobrasca
1
1-76839
1 day ago
105-83937
105 days ago
13-72205
13 days
33323 harahu
author:harahu
doc(Algebra): fix file refs Address some stale file refs in `Algebra`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
4/3 Mathlib/Algebra/Group/Pointwise/Finset/Interval.lean,Mathlib/Algebra/Module/Submodule/Lattice.lean,Mathlib/Algebra/Order/Module/OrderedSMul.lean 3 5 ['euprunin', 'github-actions', 'harahu', 'mathlib4-merge-conflict-bot'] nobody 1
1-68122
1 day ago
2-16798
2 days ago
5-34940
5 days
33028 bjornsolheim
author:bjornsolheim
feat(Geometry/Convex/Cone): minimal and maximal cone tensor products are commutative Prove that the minimal and maximal cone tensor products are commutative. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-convex-geometry 62/0 Mathlib/Geometry/Convex/Cone/TensorProduct.lean,Mathlib/LinearAlgebra/Dual/Lemmas.lean 2 13 ['artie2000', 'bjornsolheim', 'github-actions'] nobody 1
1-67703
1 day ago
1-60419
1 day ago
27-23982
27 days
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 - [x] depends on: #28853 (for simplicity) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-differential-geometry maintainer-merge 192/21 Mathlib/Analysis/Calculus/ContDiff/Basic.lean,Mathlib/Geometry/Manifold/ContMDiff/Atlas.lean,Mathlib/Geometry/Manifold/Immersion.lean,Mathlib/Geometry/Manifold/IsManifold/ExtChartAt.lean,Mathlib/Geometry/Manifold/LocalSourceTargetProperty.lean,Mathlib/Geometry/Manifold/SmoothEmbedding.lean 6 45 ['chrisflav', 'github-actions', 'grunweg', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] PatrickMassot
assignee:PatrickMassot
1
1-57567
1 day ago
2-78953
2 days ago
24-68813
24 days
33857 euprunin
author:euprunin
chore: golf and reduce compilation time --- Trace profiling results (shown if ≥10 ms before or after): * `Finset.prod_ite_mem_eq`: 38 ms before, 16 ms after 🎉 * `Finset.prod_eq_ite`: 82 ms before, 38 ms after 🎉 * `Finset.prod_dite_of_true`: 69 ms before, 30 ms after 🎉 * `Subgroup.forall_mem_sup`: 268 ms before, 51 ms after 🎉 * `Finset.nsmul_piAntidiag`: 277 ms before, 167 ms after 🎉 * `not_mulDissociated`: 642 ms before, 48 ms after 🎉 * `Finset.mem_falling`: 126 ms before, 35 ms after 🎉 * `Finset.image_diag`: 66 ms before, 44 ms after 🎉 * `Finset.biUnion_congr`: 241 ms before, 110 ms after 🎉 * `List.countP_erase`: 197 ms before, 136 ms after 🎉 * `List.triplewise_cons`: 209 ms before, 25 ms after 🎉 * `List.triplewise_append`: 298 ms before, 47 ms after 🎉 * `Nat.primeFactors_gcd`: 77 ms before, 32 ms after 🎉 * `Prod.swap_eq_iff_eq_swap`: 148 ms before, 12 ms after 🎉 * `Set.encard_eq_four`: 1034 ms before, 962 ms after 🎉 * `Set.forall_mem_image2`: 376 ms before, 33 ms after 🎉 * `Set.exists_mem_image2`: 386 ms before, 82 ms after 🎉 * `Set.pairwise_union`: 1219 ms before, 182 ms after 🎉 * `SubMulAction.mem_ofFixingSubgroup_insert_iff`: 310 ms before, 61 ms after 🎉 * `vectorSpan_add_self`: 1727 ms before, 180 ms after 🎉 * `Submodule.mem_sSup_iff_exists_finset`: 1233 ms before, 315 ms after 🎉 * `Matrix.kroneckerMap_single_single`: 436 ms before, 179 ms after 🎉 * `MeasureTheory.integral_biUnion_eq_sum_powerset`: 550 ms before, 247 ms after 🎉 * `NumberField.mixedEmbedding.fundamentalCone.card_isPrincipal_dvd_norm_le`: 945 ms before, 266 ms after 🎉 * `Set.inl_compl_union_inr_compl`: 263 ms before, 167 ms after 🎉 * `Set.ssubset_iff_sdiff_singleton`: 345 ms before, 78 ms after 🎉 * `Sublattice.le_pi`: 398 ms before, 189 ms after 🎉 * `ProbabilityTheory.Kernel.comapRight_compProd_id_prod`: 250 ms before, 145 ms after 🎉 * `Algebra.adjoin_singleton_induction`: 48 ms before, 22 ms after 🎉 * `Ideal.IsPrime.mul_mem_left_iff`: 146 ms before, 141 ms after 🎉 * `Dense.ciSup'`: 277 ms before, 150 ms after 🎉 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 28/34 Mathlib/Algebra/BigOperators/Group/Finset/Basic.lean,Mathlib/Algebra/BigOperators/Group/Finset/Piecewise.lean,Mathlib/Algebra/Group/Subgroup/Lattice.lean,Mathlib/Algebra/Order/Antidiag/Pi.lean,Mathlib/Combinatorics/Additive/Dissociation.lean,Mathlib/Combinatorics/SetFamily/LYM.lean,Mathlib/Data/Finset/Prod.lean,Mathlib/Data/Finset/Union.lean,Mathlib/Data/List/Count.lean,Mathlib/Data/Nat/PrimeFin.lean,Mathlib/Data/Set/Card.lean,Mathlib/Data/Set/NAry.lean,Mathlib/Data/Set/Pairwise/Basic.lean,Mathlib/GroupTheory/GroupAction/SubMulAction/OfFixingSubgroup.lean,Mathlib/LinearAlgebra/AffineSpace/AffineSubspace/Defs.lean,Mathlib/LinearAlgebra/Finsupp/Span.lean,Mathlib/LinearAlgebra/Matrix/Kronecker.lean,Mathlib/MeasureTheory/Integral/Bochner/Set.lean,Mathlib/NumberTheory/NumberField/CanonicalEmbedding/FundamentalCone.lean,Mathlib/Order/BooleanAlgebra/Set.lean,Mathlib/Order/Sublattice.lean,Mathlib/Probability/Kernel/Composition/CompProd.lean,Mathlib/RingTheory/Adjoin/Polynomial.lean,Mathlib/RingTheory/Ideal/Prime.lean,Mathlib/Topology/Order/IsLUB.lean 25 4 ['euprunin', 'github-actions', 'harahu', 'leanprover-radar', 'mathlib4-merge-conflict-bot'] nobody 1
1-43638
1 day ago
1-28898
1 day ago
3-15326
3 days
33388 plby
author:plby
doc(docs/100.yaml): add recently-proven theorems Two theorems from Freek Wiedijk's list of 100 theorems are currently in a Mathlib PR in progress. Five theorems from the list have been auto-formalized by Aristotle from Harmonic, and their solutions are hosted elsewhere. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict new-contributor awaiting-author 43/1 docs/100.yaml,docs/1000.yaml 2 26 ['Ruben-VandeVelde', 'github-actions', 'jcommelin', 'jsm28', 'mathlib4-merge-conflict-bot', 'mo271', 'ocfnash', 'plby', 'wwylele'] jcommelin, kim-em, ocfnash
assignee:kim-em assignee:jcommelin assignee:ocfnash
1
1-4233
1 day ago
7-70272
7 days ago
6-74167
6 days
33765 JovanGerb
author:JovanGerb
feat(Order/CompleteLattice/Defs): `to_dual` for `CompleteSemilattice`s This PR uses `to_dual` for `CompleteSemilatticeSup` and `CompleteSemilatticeInf`. These will need to be refactored/deprecated in the future, but I think it makes sense to make the code smaller (using `to_dual`) before such a refactor. --- - [ ] depends on: #33760 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR large-import t-order 157/360 Mathlib/Order/Bounds/Basic.lean,Mathlib/Order/Bounds/Defs.lean,Mathlib/Order/CompleteLattice/Defs.lean,Mathlib/Order/Interval/Set/Defs.lean,Mathlib/Tactic/Translate/ToDual.lean 5 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'vihdzp'] nobody 1
1-3550
1 day ago
unknown
unknown
33939 mitchell-horner
author:mitchell-horner
chore(Analysis/Normed): redefine `seminormFromConst'` without `choose` Redefine `seminormFromConst'` using `iInf` instead of `choose`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 136/94 Mathlib.lean,Mathlib/Analysis/Normed/Unbundled/SeminormFromConst.lean,Mathlib/Analysis/Normed/Unbundled/SpectralNorm.lean,Mathlib/Topology/Instances/NNReal/Lemmas.lean,Mathlib/Topology/Instances/Real/Lemmas.lean,Mathlib/Topology/Instances/Real/Periodic.lean 6 14 ['github-actions', 'mitchell-horner', 'vihdzp'] nobody 1
0-81918
22 hours ago
0-84502
23 hours ago
1-10203
1 day
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? [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) delegated t-meta 55/14 Mathlib/Tactic/Abel.lean,Mathlib/Tactic/FieldSimp.lean,Mathlib/Tactic/Ring/RingNF.lean,Mathlib/Util/AtomM/Recurse.lean,MathlibTest/FieldSimp.lean 5 29 ['FLDutchmann', 'JovanGerb', 'Vierkantor', 'github-actions', 'grunweg', 'leanprover-radar', 'mathlib-bors'] alexjbest
assignee:alexjbest
2
0-78359
21 hours ago
0-78359
21 hours ago
26-19830
26 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. The violations found by this linter are fixed in #33068 (merged) and #33148 (merged). Note that the portion of this diff corresponding to the actual linter file is relatively small (+68 -11), and is very similar to the `unusedDecidableInType` linter. The majority of the diff in the linter file itself is factoring out the workaround to lean4#11313 (which is used in both linters); the rest of the diff comes from reorganizing tests and adding tests. --- - [x] depends on: #31142 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) maintainer-merge file-removed 304/46 Mathlib/Tactic/Linter/UnusedInstancesInType.lean,MathlibTest/UnusedInstancesInType/Basic.lean,MathlibTest/UnusedInstancesInType/Decidable.lean,MathlibTest/UnusedInstancesInType/Fintype.lean,MathlibTest/UnusedInstancesInType/FintypeNeedingImport.lean,MathlibTest/UnusedInstancesInType/SetOption.lean 6 15 ['JovanGerb', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'thorimur'] JovanGerb
assignee:JovanGerb
1
0-62542
17 hours ago
2-48797
2 days ago
40-21713
40 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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra awaiting-author
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 31 ['github-actions', 'joelriou', 'kckennylau', 'llllvvuu', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] joelriou
assignee:joelriou
1
0-58008
16 hours ago
57-5544
57 days ago
20-28643
20 days
33919 tb65536
author:tb65536
feat(Algebra/Polynomial/Roots): Action of group on `rootSet` This PR adds an instance for `MulAction G (f.rootSet R)` whenever a `MulSemiringAction G R` satisfies `SMulCommClass G S R`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-ring-theory t-algebra delegated
label:t-algebra$
43/1 Mathlib/Algebra/Polynomial/AlgebraMap.lean,Mathlib/Algebra/Polynomial/Roots.lean 2 11 ['alreadydone', 'eric-wieser', 'github-actions', 'mathlib-bors', 'tb65536'] nobody 1
0-57480
15 hours ago
0-64607
17 hours ago
0-74129
20 hours
33972 YuvalFilmus
author:YuvalFilmus
feat(Analysis/Polynomial/Order): polynomial has fixed sign beyond largest root We prove that a polynomial has fixed sign beyond its largest root. One could also prove similar results about the smallest root, but they will be more awkward since they will depend on the parity of the (natural) degree; suggestions welcome (perhaps for a future PR). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis 73/0 Mathlib.lean,Mathlib/Analysis/Polynomial/Order.lean 2 6 ['YuvalFilmus', 'github-actions', 'vihdzp'] nobody 1
0-6529
1 hour ago
0-37198
10 hours ago
0-6812
1 hour
33909 YaelDillies
author:YaelDillies
feat(SetTheory/Cardinal): more lemmas about `ENat` and deduplicate a few pairs. From ProofBench --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-set-theory 79/49 Mathlib/Data/Finite/Card.lean,Mathlib/Data/Set/Card.lean,Mathlib/FieldTheory/CardinalEmb.lean,Mathlib/LinearAlgebra/Matrix/Rank.lean,Mathlib/RingTheory/Length.lean,Mathlib/SetTheory/Cardinal/ENat.lean,Mathlib/SetTheory/Cardinal/Finite.lean,Mathlib/SetTheory/Cardinal/NatCount.lean,Mathlib/SetTheory/Cardinal/ToNat.lean 9 2 ['github-actions', 'vihdzp'] nobody 1
0-2935
48 minutes ago
unknown
unknown
32882 DavidLedvinka
author:DavidLedvinka
feat(Probability): add `Adapted ` Add `Adapted` which is a version of `StronglyAdapted` for `Measurable `rather than `StronglyMeasurable`. Also add theorems which state when one property implies the other and when they are equivalent. - [x] depends on: #33063 t-measure-probability delegated 65/95 Mathlib/Probability/Kernel/Disintegration/Density.lean,Mathlib/Probability/Martingale/BorelCantelli.lean,Mathlib/Probability/Martingale/Centering.lean,Mathlib/Probability/Martingale/Upcrossing.lean,Mathlib/Probability/Process/Adapted.lean,Mathlib/Probability/Process/Stopping.lean 6 8 ['DavidLedvinka', 'RemyDegenne', 'github-actions', 'kex-y', 'mathlib-bors', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] kex-y
assignee:kex-y
1
0-1909
31 minutes ago
0-1909
28 minutes ago
3-24094
3 days
33390 farmanb
author:farmanb
feat(RingTheory/Ideal): generalize Submodule.colon to sets This PR generalizes `Submodule.colon` to arguments of type `Set M` in the second slot and updates the surrounding API accordingly. Main changes * Generalize `Submodule.colon` to take `S : Set M` rather than `P : Submodule R M`. * Normalize theorems/lemmas to use `Set.univ` instead of `⊤` where appropriate. * Strengthen `iInf_colon_iSup` by removing an unnecessary commutativity assumption. * Update monotonicity and inclusion lemmas (e.g. `_root_.Ideal.le_colon`) to use set inclusions. * Add `colon_bot'` (`CommSemiring`): identify `⊥.colon S` with the annihilator of `Submodule.span R S`. * Adjust annihilator-related proofs to account for the generalized colon, using explicit coercions such as `Submodule.top_coe`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-ring-theory new-contributor 113/54 Mathlib/RingTheory/Ideal/Colon.lean,Mathlib/RingTheory/Ideal/Oka.lean,Mathlib/RingTheory/Lasker.lean,Mathlib/RingTheory/Noetherian/OfPrime.lean,Mathlib/RingTheory/PrincipalIdealDomainOfPrime.lean,Mathlib/RingTheory/Support.lean 6 67 ['erdOne', 'farmanb', 'github-actions', 'tb65536'] nobody 1
0-737
12 minutes ago
0-20533
5 hours ago
4-59904
4 days
33920 Citronhat
author:Citronhat
feat(topology): generalize tendsto_inv_iff from ℝ≥0∞ to topological groups This PR implements the [TODO](https://github.com/leanprover-community/mathlib4/blob/b2f24e70b375e42e5a60251a2f43baa20ca668f1/Mathlib/Topology/Instances/ENNReal/Lemmas.lean#L468C1-L471C70) in `Topology.Instances.ENNReal.Lemmas` by moving the lemma to a more general setting. - Add a general lemma `tendsto_inv_iff` in `Topology.Algebra.Group.Basic` (with `@[simp]`), whose proof is the same as the previous `ℝ≥0∞` proof, just stated for an arbitrary `G` with `[InvolutiveInv G]` and `[ContinuousInv G]`. - Mark it `@[to_additive (attr := simp)]`, so the additive analogue is generated automatically. - Change `ENNReal.tendsto_inv_iff` in `Topology.Instances.ENNReal.Lemmas` to be a wrapper around the new lemma, preserving the existing statement/attributes and avoiding duplication. No mathematical content changes: this is a relocation/generalization of the existing proof plus the additive version. t-topology new-contributor 11/9 Mathlib/MeasureTheory/Covering/Differentiation.lean,Mathlib/MeasureTheory/Integral/Lebesgue/Markov.lean,Mathlib/Topology/Algebra/Group/Basic.lean,Mathlib/Topology/Instances/ENNReal/Lemmas.lean 4 4 ['Citronhat', 'github-actions', 'vihdzp'] nobody 1
0-497
8 minutes ago
0-3876
1 hour ago
1-35816
1 day
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). --- - [x] depends on: #31205 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis t-convex-geometry ready-to-merge 62/0 Mathlib/Analysis/Convex/Side.lean 1 4 ['YaelDillies', 'github-actions', 'jcommelin', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] YaelDillies
assignee:YaelDillies
1
0-477
7 minutes ago
0-478
4 minutes ago
37-85221
37 days

All open PRs

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
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-algebra
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
533-5311
1 year ago
unknown
unknown
14889 yuma-mizuno
author:yuma-mizuno
feat(CategoryTheory/Bicategory/Monad): define monad in bicategory --- - [ ] depends on: #12107 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP blocked-by-other-PR t-category-theory 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
533-5311
1 year ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-algebra t-algebraic-geometry
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
533-5310
1 year ago
unknown
unknown
14036 adomani
author:adomani
Test/decl diff in lean --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
533-5310
1 year ago
unknown
unknown
14167 alreadydone
author:alreadydone
feat: Group scheme structure on Weierstrass curve --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-algebraic-geometry workshop-AIM-AG-2024 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
533-5310
1 year ago
unknown
unknown
12952 adomani
author:adomani
test: length statistics --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP test-ci 124/0 .github/workflows/mathlib_stats.yml,.github/workflows/ml_stats_label.yaml,scripts/mathlib_stats.sh 3 9 ['github-actions'] nobody
533-5309
1 year ago
unknown
unknown
13297 urkud
author:urkud
feat(Semicontinuous): add `comp` lemma --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-topology t-order 31/13 Mathlib/Topology/Semicontinuous.lean 1 3 ['sgouezel', 'urkud'] nobody
533-5309
1 year ago
unknown
unknown
13372 adomani
author:adomani
dev: generic replacement --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
533-5309
1 year ago
unknown
unknown
13512 adomani
author:adomani
test: count all --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
533-5309
1 year ago
unknown
unknown
12416 adomani
author:adomani
chore: remove some cdots --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
533-5308
1 year ago
unknown
unknown
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
533-5308
1 year ago
unknown
unknown
12473 adomani
author:adomani
first translations --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
533-5308
1 year ago
unknown
unknown
12528 adomani
author:adomani
test: autotranslations Bot --> Top --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
533-5308
1 year ago
unknown
unknown
12588 adomani
author:adomani
remove trailingDegree --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
533-5308
1 year ago
unknown
unknown
12608 eric-wieser
author:eric-wieser
feat: allow `nsmul` / `zsmul` to be omitted again, with a warning --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-algebra t-meta
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
533-5308
1 year ago
unknown
unknown
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`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra t-meta
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
533-5308
1 year ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP 57/14 Mathlib/NumberTheory/RamificationInertia.lean 1 3 ['MichaelStollBayreuth', 'github-actions', 'leanprover-bot'] nobody
533-5308
1 year ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-linter tech debt 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
533-5308
1 year ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
533-5308
1 year ago
unknown
unknown
12984 adomani
author:adomani
Adomani/periodic reports dev custom action --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP test-ci 366/0 .github/workflows/mathlib_stats.yml,.github/workflows/ml_stats_label.yaml,scripts/count_decls.lean,scripts/mathlib_stats.sh 4 69 ['github-actions'] nobody
533-5308
1 year ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra t-number-theory 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
533-5308
1 year ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-logic 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
533-5307
1 year ago
unknown
unknown
12192 Ruben-VandeVelde
author:Ruben-VandeVelde
feat: generalize isLittleO_const_id_atTop/atBot From PNT+. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-analysis 10/4 Mathlib/Analysis/Asymptotics/Asymptotics.lean 1 6 ['Ruben-VandeVelde', 'llllvvuu', 'urkud'] nobody
533-5307
1 year ago
unknown
unknown
10024 ADedecker
author:ADedecker
feat: rename `connectedComponentOfOne` to `identityComponent`, prove that it is normal and open --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-topology awaiting-CI 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
533-5306
1 year ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-analysis 58/42 Mathlib/Analysis/NormedSpace/BoundedLinearMaps.lean 1 3 ['github-actions', 'j-loreaux', 'urkud'] nobody
533-5306
1 year ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-meta 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
533-5306
1 year ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-order t-logic 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
533-5306
1 year ago
unknown
unknown
10842 mcdoll
author:mcdoll
chore: simplify proofs using new positivity extensions and tests --- - [x] depends on: #10661 - [ ] depends on: #10796 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP blocked-by-other-PR 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
533-5306
1 year ago
unknown
unknown
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP RFC t-category-theory 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
533-5306
1 year ago
unknown
unknown
11100 eric-wieser
author:eric-wieser
feat(CategoryTheory/Limits): add `Functor.mapBinaryBiconeInv` --- - [ ] depends on: #11130 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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 merge-conflict t-category-theory awaiting-CI 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
533-5306
1 year ago
unknown
unknown
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-meta 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
533-5305
1 year ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-algebra
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
533-5305
1 year ago
unknown
unknown
8582 eric-wieser
author:eric-wieser
wip --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
533-5305
1 year ago
unknown
unknown
8616 eric-wieser
author:eric-wieser
feat(Algebra/FreeAlgebra): add right action and `IsCentralScalar` --- - [ ] depends on: #8652 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra awaiting-CI
label:t-algebra$
30/8 Mathlib/Algebra/FreeAlgebra.lean 1 1 ['leanprover-community-mathlib4-bot'] nobody
533-5305
1 year ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-algebra
label:t-algebra$
80/18 Mathlib/GroupTheory/Congruence.lean,Mathlib/RingTheory/Congruence.lean 2 6 ['YaelDillies', 'eric-wieser'] nobody
533-5305
1 year ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra
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
533-5305
1 year ago
unknown
unknown
8906 jjaassoonn
author:jjaassoonn
feat: add some missing lemmas about linear algebra --- - [ ] depends on: #8905 [lifting injective modules to higher universe] [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-algebra
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
533-5305
1 year ago
unknown
unknown
8961 eric-wieser
author:eric-wieser
refactor: use the coinduced topology on ULift --- - [x] depends on: #8958 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) please-adopt merge-conflict awaiting-author awaiting-CI 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
533-5305
1 year ago
unknown
unknown
9146 laughinggas
author:laughinggas
feat(Data/ZMod/Defs): Topological structure on `ZMod` Added a discrete topology structure to `ZMod n` for all `n` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra awaiting-author t-topology
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
533-5305
1 year ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-algebra
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
533-5305
1 year ago
unknown
unknown
9252 astrainfinita
author:astrainfinita
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-algebra t-order merge-conflict slow-typeclass-synthesis awaiting-author
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 ['astrainfinita', 'leanprover-bot', 'urkud'] nobody
533-5305
1 year ago
unknown
unknown
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) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-analysis 540/0 Mathlib.lean,Mathlib/Analysis/Convex/ConvexFunction.lean 2 15 ['github-actions', 'winstonyin'] nobody
533-5305
1 year ago
unknown
unknown
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" [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-meta 24/0 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Common.lean,Mathlib/Tactic/TryAssumption.lean 4 5 ['alexjbest', 'j-loreaux', 'jcommelin'] nobody
533-5305
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-analysis 71/0 Mathlib/Analysis/Complex/AbsMax.lean 1 8 ['dupuisf', 'j-loreaux'] nobody
533-5305
1 year ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-category-theory 21/8 Mathlib/Algebra/Category/ModuleCat/Adjunctions.lean,Mathlib/CategoryTheory/Monoidal/Functorial.lean,Mathlib/CategoryTheory/Monoidal/Limits.lean 3 0 [] nobody
533-5305
1 year ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-algebra t-measure-probability merge-conflict t-analysis
label:t-algebra$
97/0 Mathlib/Analysis/NormedSpace/TrivSqZeroExt.lean 1 7 ['github-actions', 'leanprover-community-mathlib4-bot'] nobody
533-5305
1 year ago
unknown
unknown
9504 alreadydone
author:alreadydone
chore: remove some IsSeparable assumptions --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-algebra
label:t-algebra$
41/14 Mathlib/NumberTheory/NumberField/Norm.lean,Mathlib/RingTheory/Norm.lean 2 0 [] nobody
533-5305
1 year ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-algebra t-analysis awaiting-CI
label:t-algebra$
119/0 Mathlib/Analysis/Calculus/DualNumber.lean 1 4 ['github-actions'] nobody
533-5305
1 year ago
unknown
unknown
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`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-algebra awaiting-CI
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
533-5305
1 year ago
unknown
unknown
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`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) I will write a longer PR description for this once CI is happy WIP merge-conflict awaiting-author help-wanted t-analysis 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
533-5305
1 year ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
533-5304
1 year ago
unknown
unknown
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` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-algebra
label:t-algebra$
31/0 Mathlib/LinearAlgebra/Matrix/Spectrum.lean 1 0 [] nobody
533-5304
1 year ago
unknown
unknown
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') ``` [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
533-5304
1 year ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author help-wanted awaiting-CI 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
533-5304
1 year ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-meta 327/0 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/ResynthInstances.lean,test/ResynthInstances.lean 4 0 [] nobody
533-5304
1 year ago
unknown
unknown
6931 urkud
author:urkud
refactor(Analysis/Normed*): use `RingHomIsometric` for `*.norm_cast` --- I don't understand why linter fails. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict help-wanted t-analysis 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
533-5304
1 year ago
unknown
unknown
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 ![00HD](https://stacks.math.columbia.edu/tag/00HD) 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 ---------- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
533-5304
1 year ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-meta 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
533-5304
1 year ago
unknown
unknown
7351 shuxuezhuyi
author:shuxuezhuyi
feat(Topology/Algebra/Order): extend function on `Ioo` to `Icc` Extend a strictly monotone function defined on an open interval. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-order 59/0 Mathlib.lean,Mathlib/Data/Set/Function.lean,Mathlib/Topology/Algebra/Order/IccExtendFromIoo.lean 3 7 ['j-loreaux', 'shuxuezhuyi'] nobody
533-5304
1 year ago
unknown
unknown
7467 ADedecker
author:ADedecker
feat: spectrum of X →ᵇ ℂ is StoneCech X --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-analysis 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
533-5304
1 year ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP blocked-by-core-PR blocked-by-other-PR merge-conflict t-meta 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
533-5304
1 year ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-topology blocked-by-other-PR 162/0 Mathlib.lean,Mathlib/Topology/Algebra/Order/IccExtendFromIoo.lean 2 1 ['leanprover-community-mathlib4-bot'] nobody
533-5304
1 year ago
unknown
unknown
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 ``` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-algebra t-meta
label:t-algebra$
257/48 Mathlib/Tactic/Ring/Basic.lean,test/linear_combination.lean,test/ring.lean 3 1 ['eric-wieser'] nobody
533-5304
1 year ago
unknown
unknown
7615 eric-wieser
author:eric-wieser
chore(LinearAlgebra/Basic): generalize compatibleMaps to semilinear maps Spotted while reviewing #7611 --- - [x] depends on: #7611 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra easy awaiting-CI
label:t-algebra$
9/33 Mathlib/LinearAlgebra/Basic.lean 1 1 ['leanprover-community-mathlib4-bot'] nobody
533-5304
1 year ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-measure-probability 53/1 Mathlib/MeasureTheory/Measure/MutuallySingular.lean,lean-toolchain 2 6 ['RemyDegenne', 'digama0', 'eric-wieser', 'fpvandoorn'] nobody
533-5304
1 year ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-algebra
label:t-algebra$
52/0 Mathlib/LinearAlgebra/Matrix/ProjectiveSpecialLinearGroup.lean 1 3 ['jcommelin', 'leanprover-community-mathlib4-bot', 'shuxuezhuyi'] jcommelin
assignee:jcommelin
533-5304
1 year ago
unknown
unknown
7875 astrainfinita
author:astrainfinita
chore: make `SMulCommClass A A B` and `SMulCommClass A B B` higher priority --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict slow-typeclass-synthesis t-algebra
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
533-5304
1 year ago
unknown
unknown
7909 mcdoll
author:mcdoll
fix(Tactic/Continuity): remove npowRec and add new tag for Continuous.pow --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-topology t-meta 14/9 Mathlib/Tactic/Continuity.lean,Mathlib/Topology/Category/TopCat/Limits/Basic.lean,test/Continuity.lean 3 2 ['eric-wieser'] nobody
533-5304
1 year ago
unknown
unknown
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]`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra awaiting-CI
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
533-5304
1 year ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-algebra
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
533-5304
1 year ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR t-meta 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
533-5304
1 year ago
unknown
unknown
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
533-5303
1 year ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-meta 482/1 Mathlib/Tactic/Backtracking.lean,test/Backtracking.lean 2 0 [] nobody
533-5303
1 year ago
unknown
unknown
4775 thorimur
author:thorimur
feat: `SubExpr` utilities This file contains utilities for handling positions in expressions, including folding over subexpressions along with their positions. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-meta 148/0 Mathlib.lean,Mathlib/Lean/SubExpr.lean 2 0 [] nobody
533-5303
1 year ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR t-meta 491/1 Mathlib.lean,Mathlib/Lean/Meta/AppBuilder.lean,Mathlib/Lean/Meta/Basic.lean,Mathlib/Lean/Meta/ExprWithLevels.lean 4 1 ['kim-em'] nobody
533-5303
1 year ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra awaiting-CI
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
533-5303
1 year ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-algebra
label:t-algebra$
110/55 Mathlib/FieldTheory/Adjoin.lean 1 0 [] nobody
533-5303
1 year ago
unknown
unknown
5912 ADedecker
author:ADedecker
feat(Analysis.Distribution.ContDiffMapSupportedIn): space of smooth maps with support in a fixed compact --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-analysis 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
533-5303
1 year ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-analysis 26/0 Mathlib/Analysis/SpecialFunctions/Gaussian.lean 1 3 ['ocfnash', 'slerpyyy', 'urkud'] nobody
533-5303
1 year ago
unknown
unknown
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) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-CI 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
533-5303
1 year ago
unknown
unknown
6195 eric-wieser
author:eric-wieser
chore(RingTheory/TensorProduct): golf the `mul` definition --- - [x] depends on: #6211 - [x] depends on: #6187 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) Strangely this causes a timeout downstream merge-conflict t-algebra awaiting-CI
label:t-algebra$
4/29 Mathlib/RingTheory/TensorProduct.lean 1 1 ['leanprover-community-mathlib4-bot'] nobody
533-5303
1 year ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-algebra t-analysis
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
533-5303
1 year ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-category-theory 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
533-5303
1 year ago
unknown
unknown
6328 astrainfinita
author:astrainfinita
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-algebra awaiting-CI
label:t-algebra$
14/14 Mathlib/RingTheory/NonUnitalSubsemiring/Basic.lean,Mathlib/RingTheory/Subsemiring/Basic.lean,lean-toolchain 3 1 ['digama0'] nobody
533-5303
1 year ago
unknown
unknown
6330 astrainfinita
author:astrainfinita
chore: make some instance about `Sub...Class` higher priority than `Sub...` The opposite direction to #6328. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-algebra slow-typeclass-synthesis
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
533-5303
1 year ago
unknown
unknown
6403 astrainfinita
author:astrainfinita
chore: change instance priorities of `Ordered*` hierarchy --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-order merge-conflict slow-typeclass-synthesis 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
533-5303
1 year ago
unknown
unknown
6491 eric-wieser
author:eric-wieser
chore(Mathlib/Algebra/Hom/GroupAction): add `SMulHomClass.comp_smul` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra
label:t-algebra$
24/10 Mathlib/Algebra/Hom/GroupAction.lean 1 0 [] nobody
533-5303
1 year ago
unknown
unknown
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. merge-conflict WIP t-differential-geometry t-measure-probability 165/0 Mathlib.lean,Mathlib/Geometry/Manifold/MeasureZero.lean,docs/references.bib 3 27 ['ADedecker', 'github-actions', 'grunweg', 'mo271', 'sgouezel'] ADedecker
assignee:ADedecker
533-5303
1 year ago
unknown
unknown
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-meta 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
533-5302
1 year ago
unknown
unknown
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-meta 131/32 Mathlib/Tactic/Conv.lean,Mathlib/Tactic/NormNum/Core.lean,Mathlib/Tactic/PushNeg.lean,docs/Conv/Guide.lean 4 0 [] nobody
528-68012
1 year ago
unknown
unknown
13852 astrainfinita
author:astrainfinita
perf: skip some typeclasses in TC search --- - [ ] depends on: #7873 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict slow-typeclass-synthesis blocked-by-other-PR 45/33 Mathlib/Algebra/Group/Defs.lean,Mathlib/Algebra/Ring/Defs.lean,Mathlib/RingTheory/Norm.lean 3 21 ['MichaelStollBayreuth', 'astrainfinita', 'github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot'] nobody
528-61692
1 year ago
unknown
unknown
7903 urkud
author:urkud
feat: define `UnboundedSpace` --- The new instances generate some timeouts, and I don't understand why. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict help-wanted t-topology 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
525-79681
1 year ago
unknown
unknown
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). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-linter 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
520-72775
1 year ago
unknown
unknown
15679 adomani
author:adomani
test: refactor in CI --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
520-48857
1 year ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-topology blocked-by-other-PR t-order 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
518-85357
1 year ago
unknown
unknown
10629 madvorak
author:madvorak
feat: List.cons_sublist_append_iff_right --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-data 11/0 Mathlib/Data/List/Basic.lean 1 1 ['eric-wieser'] nobody
518-85248
1 year ago
unknown
unknown
9973 Ruben-VandeVelde
author:Ruben-VandeVelde
feat: polynomials formed by lists From https://github.com/leanprover-community/mathlib/pull/15476 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) please-adopt merge-conflict t-data 311/0 Mathlib.lean,Mathlib/Data/Polynomial/OfList.lean 2 0 [] nobody
518-84781
1 year ago
unknown
unknown
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`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-category-theory 105/0 Mathlib.lean,Mathlib/CategoryTheory/Monoidal/Induced.lean 2 3 ['eric-wieser', 'github-actions', 'joelriou'] nobody
518-83180
1 year ago
unknown
unknown
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`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-linter 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
518-69944
1 year ago
unknown
unknown
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)` [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-algebra new-contributor
label:t-algebra$
5/0 Mathlib/Algebra/Group/Basic.lean 1 3 ['eric-wieser', 'github-actions', 'kim-em'] nobody
517-84096
1 year ago
unknown
unknown
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) merge-conflict WIP t-algebra
label:t-algebra$
10/3 Mathlib/Algebra/DirectSum/Module.lean,Mathlib/LinearAlgebra/FreeModule/Basic.lean 2 1 ['github-actions'] nobody
517-81965
1 year ago
unknown
unknown
13010 ADedecker
author:ADedecker
feat: relax universe constraint in stoneCechExtend --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-topology 33/3 Mathlib/Topology/StoneCech.lean 1 2 ['ADedecker', 'erdOne'] nobody
517-81762
1 year ago
unknown
unknown
12411 adomani
author:adomani
feat: more linting of cdots --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-linter 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
517-81625
1 year ago
unknown
unknown
12279 casavaca
author:casavaca
WIP: feat: Holder's inequality n-ary --- - [x] depends on #12291 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-analysis 129/0 Mathlib/Analysis/MeanInequalities.lean,Mathlib/Analysis/SpecialFunctions/Pow/Real.lean 2 13 ['github-actions'] nobody
517-81610
1 year ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-topology 274/130 Mathlib/Analysis/BoundedVariation.lean,Mathlib/MeasureTheory/Integral/FundThmCalculus.lean,Mathlib/Order/Filter/Basic.lean,Mathlib/Topology/Semicontinuous.lean 4 0 [] nobody
517-81572
1 year ago
unknown
unknown
11520 thorimur
author:thorimur
feat: `linting_rules` and deprecated syntax --- Experimental. WIP. Might not be performance-viable. - [ ] depends on: #11519 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR t-meta 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
517-81562
1 year ago
unknown
unknown
11519 thorimur
author:thorimur
feat: `syntax_rules` --- Experimental. WIP. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-meta 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
517-81548
1 year ago
unknown
unknown
11393 mcdoll
author:mcdoll
feat(Analysis/Distribution/SchwartzSpace): The Heine-Borel property --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-analysis 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
517-81538
1 year ago
unknown
unknown
9444 erdOne
author:erdOne
feat: Various instances regarding `𝓞 K`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict help-wanted t-number-theory 27/0 Mathlib/NumberTheory/NumberField/Basic.lean,Mathlib/RingTheory/IntegralClosure.lean 2 9 ['erdOne', 'leanprover-bot', 'mattrobball', 'riccardobrasca', 'xroblot'] nobody
517-81457
1 year ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-computability 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
517-81422
1 year ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-topology 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
517-81390
1 year ago
unknown
unknown
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). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP RFC t-meta 24/0 Mathlib/Tactic/ComputeDegree.lean 1 0 [] nobody
517-81244
1 year ago
unknown
unknown
8608 eric-wieser
author:eric-wieser
feat: multiplicativize `AddTorsor` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-algebra
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
517-81067
1 year ago
unknown
unknown
9154 astrainfinita
author:astrainfinita
feat: `npow` / `nsmul` / `Nat.cast`/ `zpow` / `zsmul` implemented using `Nat.binaryRec` --- - [ ] depends on: https://github.com/leanprover/lean4/pull/3756 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-algebra 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 ['astrainfinita', 'eric-wieser', 'kim-em', 'leanprover-community-mathlib4-bot'] nobody
517-81035
1 year ago
unknown
unknown
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP CI 29/0 lakefile.lean 1 3 ['kim-em', 'tydeu'] nobody
517-81009
1 year ago
unknown
unknown
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) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) - [x] depends on: #6059 - [ ] define direct sum of cones - [ ] weak duality - [ ] regular duality - [ ] slater condition - [ ] strong duality merge-conflict WIP t-analysis 159/0 Mathlib.lean,Mathlib/Analysis/Convex/Cone/ConeLinearProgram.lean 2 1 ['leanprover-community-mathlib4-bot'] nobody
517-80954
1 year ago
unknown
unknown
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-topology 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
517-80948
1 year ago
unknown
unknown
8100 digama0
author:digama0
feat: add support for other types in norm_num --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-meta 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
517-80816
1 year ago
unknown
unknown
13163 erdOne
author:erdOne
feat(.vscode/module-docstring.code-snippet): Prevent auto-complete from firing on `do` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-meta 5/0 .vscode/module-docstring.code-snippets 1 5 ['erdOne', 'grunweg', 'robertylewis', 'trivial1711'] nobody
517-79558
1 year ago
unknown
unknown
15585 astrainfinita
author:astrainfinita
test make `HasQuotient.quotient'` reducible --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra
label:t-algebra$
8/1 Mathlib/Algebra/Quotient.lean,Mathlib/GroupTheory/Coset.lean 2 1 ['github-actions'] nobody
516-26824
1 year ago
unknown
unknown
15586 astrainfinita
author:astrainfinita
test make `HasQuotient` out put a `setoid` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra
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
516-26824
1 year ago
unknown
unknown
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`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-computability tech debt 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
514-48093
1 year ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebraic-geometry t-category-theory 210/0 Mathlib.lean,Mathlib/AlgebraicGeometry/FunctorOfPoints.lean,Mathlib/AlgebraicGeometry/OpenImmersion.lean 3 4 ['github-actions', 'grunweg', 'leanprover-community-mathlib4-bot'] nobody
514-47952
1 year ago
unknown
unknown
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`. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
514-47851
1 year ago
unknown
unknown
9978 astrainfinita
author:astrainfinita
chore(FieldTheory/KummerExtension): move some lemmas earlier --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-algebra
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
514-47643
1 year ago
unknown
unknown
12429 adomani
author:adomani
feat: toND -- auto-generating natDegree This is an experiment to automatically translate theorems about `degree` to theorems about `natDegree`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra RFC merge-conflict awaiting-author t-meta
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
514-46954
1 year ago
unknown
unknown
15823 eric-wieser
author:eric-wieser
Quotients of rings in model theory --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-logic 55/13 Mathlib/ModelTheory/Algebra/Ring/FreeCommRing.lean,Mathlib/ModelTheory/Syntax.lean 2 1 ['github-actions'] nobody
514-25517
1 year ago
unknown
unknown
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) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra
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
514-2641
1 year ago
unknown
unknown
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`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-data new-contributor 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
513-69005
1 year ago
unknown
unknown
15448 urkud
author:urkud
chore(*): deprecate `Option.elim'` Use `Option.elim` instead. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author tech debt 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
513-58058
1 year ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-data 169/3 Mathlib/Data/Setoid/Basic.lean,Mathlib/Data/Setoid/Partition.lean,Mathlib/Order/Closure.lean 3 1 ['leanprover-community-mathlib4-bot'] nobody
511-71279
1 year ago
unknown
unknown
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-algebra
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
511-71259
1 year ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-algebra
label:t-algebra$
294/0 Mathlib.lean,Mathlib/LinearAlgebra/Matrix/DFT.lean 2 26 ['MohanadAhmed', 'ericrbg'] nobody
511-71097
1 year ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra awaiting-author t-number-theory
label:t-algebra$
565/12 Mathlib/NumberTheory/EllipticDivisibilitySequence.lean 1 55 ['Multramate', 'alreadydone', 'github-actions', 'grunweg', 'leanprover-community-mathlib4-bot'] nobody
505-84701
1 year ago
unknown
unknown
15600 adomani
author:adomani
feat: lint also `let` vs `have` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-linter 77/26 Mathlib/Tactic/Linter/HaveLetLinter.lean,test/HaveLetLinter.lean 2 1 ['github-actions'] nobody
504-52977
1 year ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP awaiting-author 144/0 Mathlib/GameTheory/FairDivision/Discrete/Basic.lean 1 9 ['Shreyas4991', 'eric-wieser', 'github-actions'] nobody
503-50890
1 year ago
unknown
unknown
13970 adomani
author:adomani
feat: a linter to flag unnecessary uses of `nolint simpNF` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-linter 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
502-76191
1 year ago
unknown
unknown
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) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-linter 119/0 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter/CheckAsSorry.lean,test/CheckAsSorry.lean 4 1 ['github-actions'] nobody
502-75179
1 year ago
unknown
unknown
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`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-data new-contributor 90/0 Mathlib/Data/Nat/PartENat.lean 1 3 ['erdOne', 'github-actions', 'urkud'] nobody
500-80895
1 year ago
unknown
unknown
15121 Eloitor
author:Eloitor
feat: iff theorems for IsSplitEpi and IsSplitMono in opposite category --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-category-theory new-contributor 40/0 Mathlib/CategoryTheory/EpiMono.lean 1 3 ['github-actions', 'joelriou', 'mattrobball'] nobody
500-43840
1 year ago
unknown
unknown
15895 madvorak
author:madvorak
feat(Computability/ContextFreeGrammar): mapping between two types of nonterminal symbols --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-computability WIP 172/0 Mathlib/Computability/ContextFreeGrammar.lean 1 43 ['YaelDillies', 'github-actions', 'madvorak'] nobody
499-60633
1 year ago
unknown
unknown
14038 adomani
author:adomani
test/decl diff in lean dev --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
498-68693
1 year ago
unknown
unknown
14046 adomani
author:adomani
test: diff of declarations in lean --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
498-68693
1 year ago
unknown
unknown
12107 yuma-mizuno
author:yuma-mizuno
feat(Mathlib/Tactic/Widget/StringDiagram): support 2-morphisms in bicategories --- - [x] depends on: #11080 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-category-theory t-meta 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
493-63437
1 year ago
unknown
unknown
15925 yuma-mizuno
author:yuma-mizuno
feat(CategoryTheory/Monoida): proof producing coherence tactic --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-category-theory t-meta 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 1 ['github-actions'] nobody
493-23574
1 year ago
unknown
unknown
7861 shuxuezhuyi
author:shuxuezhuyi
feat(Geometry/Hyperbolic/UpperHalfPlane): instance IsometricSMul PSL(2, ℝ) ℍ --- - [ ] depends on: #7835 - [ ] depends on: #7791 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR t-euclidean-geometry 98/0 Mathlib.lean,Mathlib/Geometry/Hyperbolic/UpperHalfPlane/Basic.lean,Mathlib/LinearAlgebra/Matrix/ProjectiveSpecialLinearGroup.lean 3 1 ['leanprover-community-mathlib4-bot'] nobody
493-4634
1 year ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-meta 26/15 Mathlib/Tactic/CategoryTheory/BicategoryCoherence.lean,Mathlib/Tactic/CategoryTheory/Coherence.lean 2 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mergify'] nobody
492-67499
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra RFC
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
492-1930
1 year ago
unknown
unknown
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology awaiting-author t-algebra
label:t-algebra$
57/0 Mathlib/Topology/Algebra/ConstMulAction.lean 1 9 ['ADedecker', 'adri326', 'j-loreaux', 'jcommelin'] ADedecker
assignee:ADedecker
491-59491
1 year ago
unknown
unknown
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'`.​ --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-logic 50/0 Mathlib.lean,Mathlib/Logic/Function/ApiForExtend.lean 2 1 ['fpvandoorn'] nobody
491-17466
1 year ago
unknown
unknown
16658 adomani
author:adomani
add tips file --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP awaiting-author test-ci 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
487-46399
1 year ago
unknown
unknown
14078 Ruben-VandeVelde
author:Ruben-VandeVelde
feat(CI): continue after mk_all fails --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author CI 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
487-26699
1 year ago
unknown
unknown
11283 hmonroe
author:hmonroe
feat(ModelTheory/Satisfiability): define theory with independent sentence --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-logic 8/0 Mathlib/ModelTheory/Satisfiability.lean 1 2 ['fpvandoorn', 'hmonroe'] nobody
484-83653
1 year ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP 4/4 lake-manifest.json,lakefile.lean 2 1 ['github-actions'] nobody
482-72262
1 year ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-number-theory blocked-by-other-PR merge-conflict t-algebraic-geometry
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 8 ['Multramate', 'alreadydone', 'github-actions', 'leanprover-community-mathlib4-bot'] nobody
480-35227
1 year ago
unknown
unknown
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! --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-category-theory 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
478-8148
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra blocked-by-other-PR new-contributor
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
477-54899
1 year ago
unknown
unknown
17171 astrainfinita
author:astrainfinita
test extends carrier and property --- We need https://github.com/leanprover/lean4/issues/2666 ... [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
473-53241
1 year ago
unknown
unknown
7516 ADedecker
author:ADedecker
perf: use `abbrev` to prevent unifying useless data --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP 4/3 Mathlib/Topology/ContinuousFunction/Bounded.lean 1 3 ['ADedecker', 'leanprover-bot', 'mattrobball'] nobody
472-24901
1 year ago
unknown
unknown
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?" [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-linter 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
472-22908
1 year ago
unknown
unknown
17127 astrainfinita
author:astrainfinita
chore: remove global `Quotient.mk` `⟦·⟧` notation --- Merge this PR when we are ready to migrate to `QuotLike` API (#16421). [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-data 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
472-19944
1 year ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR new-contributor t-logic 300/7 Mathlib/ModelTheory/Complexity.lean,Mathlib/ModelTheory/Equivalence.lean,Mathlib/ModelTheory/Syntax.lean 3 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
469-50877
1 year ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR new-contributor t-logic 415/7 Mathlib/ModelTheory/Complexity.lean,Mathlib/ModelTheory/Equivalence.lean,Mathlib/ModelTheory/Syntax.lean 3 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
469-50877
1 year ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR new-contributor t-logic 525/7 Mathlib/ModelTheory/Complexity.lean,Mathlib/ModelTheory/Equivalence.lean,Mathlib/ModelTheory/Syntax.lean 3 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
469-50876
1 year ago
unknown
unknown
14712 astrainfinita
author:astrainfinita
perf: change instance priority and order about `OfNat` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict slow-typeclass-synthesis t-algebra 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 ['MichaelStollBayreuth', 'astrainfinita', 'eric-wieser', 'github-actions', 'j-loreaux', 'leanprover-bot', 'mathlib-bors'] nobody
465-82897
1 year ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-topology 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
464-18440
1 year ago
unknown
unknown
5995 astrainfinita
author:astrainfinita
feat: add APIs about `Quotient.choice` Some docs in this PR refer to the definition in #5576. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author RFC t-data 76/6 Mathlib/Data/Quot.lean 1 3 ['YaelDillies', 'astrainfinita', 'gebner'] eric-wieser
assignee:eric-wieser
462-65086
1 year ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-topology RFC 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
462-48749
1 year ago
unknown
unknown
14619 Command-Master
author:Command-Master
chore: Merge `Trunc` to `Squash` Remove `Trunc` and use `Squash` instead --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP new-contributor 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
460-11027
1 year ago
unknown
unknown
13156 erdOne
author:erdOne
refactor(Algebra/Module/LocalizedModule): Redefine `LocalizedModule` in terms of `OreLocalization`. --- - [x] depends on: #13151 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra
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
457-72226
1 year ago
unknown
unknown
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-topology t-order 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
457-71850
1 year ago
unknown
unknown
13965 pechersky
author:pechersky
feat(Data/DigitExpansion): reals via digit expansion are complete --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) - [ ] depends on: #13964 merge-conflict blocked-by-other-PR t-data 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
456-22618
1 year ago
unknown
unknown
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) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-linter 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
455-45532
1 year ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-meta 158/35 Mathlib/Tactic/Module.lean,test/module.lean 2 1 ['github-actions'] nobody
454-7890
1 year ago
unknown
unknown
10796 mcdoll
author:mcdoll
feat(Tactic/Positivity): non-negativity of functions --- This makes the `Finset.sum` and `integral_nonneg` extensions even more useful. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-meta 27/0 Mathlib/Tactic/Positivity/Core.lean 1 1 ['YaelDillies'] nobody
452-4472
1 year ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR t-data new-contributor merge-conflict awaiting-author 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
451-73534
1 year ago
unknown
unknown
12414 adomani
author:adomani
test: lint and unlint `·` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
449-70075
1 year ago
unknown
unknown
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`? [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-combinatorics new-contributor 24/0 Mathlib/Combinatorics/SimpleGraph/Map/Finite.lean 1 11 ['awueth', 'github-actions', 'jcommelin', 'kim-em', 'urkud'] nobody
449-62842
1 year ago
unknown
unknown
16925 YnirPaz
author:YnirPaz
feat(SetTheory/Cardinal/Cofinality): aleph index of singular cardinal has infinite cofinality Prove `Ordinal.aleph0_le_cof_of_not_isRegular`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-set-theory 6/0 Mathlib/SetTheory/Cardinal/Cofinality.lean 1 4 ['YnirPaz', 'github-actions', 'vihdzp'] nobody
448-41657
1 year ago
unknown
unknown
16647 eric-wieser
author:eric-wieser
feat: partitions of lists The length of this list is the bell numbers. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-combinatorics t-data 311/0 Mathlib.lean,Mathlib/Data/List/Partition.lean 2 1 ['github-actions'] nobody
447-4149
1 year ago
unknown
unknown
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. please-adopt t-data new-contributor merge-conflict 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
441-44844
1 year ago
unknown
unknown
13514 madvorak
author:madvorak
feat(Computability/ContextFreeGrammar): closure under union - [ ] depends on: #15895 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-computability blocked-by-other-PR 448/4 Mathlib/Computability/ContextFreeGrammar.lean 1 50 ['Rida-Hamadani', 'YaelDillies', 'github-actions', 'leanprover-community-mathlib4-bot', 'madvorak'] nobody
438-84862
1 year ago
unknown
unknown
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 merge-conflict t-linter blocked-by-other-PR awaiting-zulip 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
438-57595
1 year ago
unknown
unknown
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). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-meta 125/18 Mathlib/Tactic/WLOG.lean,test/wlog.lean 2 2 ['thorimur', 'urkud'] nobody
437-31501
1 year ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-meta 63/9 Mathlib/Lean/Meta.lean,Mathlib/Tactic/MkIffOfInductiveProp.lean,test/MkIffOfInductive.lean 3 6 ['Vierkantor', 'github-actions', 'urkud'] nobody
437-31255
1 year ago
unknown
unknown
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`). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-order 324/0 Mathlib.lean,Mathlib/Data/Ordering/Dickson.lean,scripts/noshake.json 3 9 ['AntoineChambert-Loir', 'b-mehta', 'github-actions'] nobody
437-9812
1 year ago
unknown
unknown
16355 Ruben-VandeVelde
author:Ruben-VandeVelde
feat: odd_{add,sub}_one --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra awaiting-author t-number-theory
label:t-algebra$
12/0 Mathlib/Algebra/Ring/Int.lean,Mathlib/Algebra/Ring/Parity.lean 2 4 ['Ruben-VandeVelde', 'github-actions', 'urkud'] nobody
436-44009
1 year ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP awaiting-author 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
436-34763
1 year ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-algebra
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
435-70222
1 year ago
unknown
unknown
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]`. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra t-order new-contributor
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
435-15410
1 year ago
unknown
unknown
18636 adomani
author:adomani
Test/latest import report dev This PR is a test accompanying #18631. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict CI 147/0 .github/workflows/latest_import.yml,lakefile.lean 2 1 ['github-actions'] nobody
434-2681
1 year ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author new-contributor t-logic 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
432-57931
1 year ago
unknown
unknown
18716 jjaassoonn
author:jjaassoonn
feat(Algebra/Module/GradedModule): quotient and subgrading - [ ] depends on: #9820 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-algebra blocked-by-other-PR awaiting-CI merge-conflict
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
432-57562
1 year ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-differential-geometry 45/0 Mathlib/Geometry/Manifold/IntegralCurve.lean,Mathlib/Topology/Algebra/Module/Basic.lean 2 9 ['github-actions', 'grunweg', 'leanprover-community-mathlib4-bot', 'winstonyin'] nobody
429-23354
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) merge-conflict awaiting-author new-contributor t-logic 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
428-10363
1 year ago
unknown
unknown
17675 astrainfinita
author:astrainfinita
perf: do not search algebraic hierarchy when searching `FunLike` hierarchy --- Unification is still very slow. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict slow-typeclass-synthesis t-algebra
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 ['astrainfinita', 'github-actions', 'leanprover-bot'] nobody
427-71896
1 year ago
unknown
unknown
9344 erdOne
author:erdOne
feat: Add `AddGroup.FG` -> `Module.Finite ℤ` as instances --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-algebra
label:t-algebra$
4/0 Mathlib/RingTheory/Finiteness.lean 1 4 ['alreadydone', 'erdOne', 'leanprover-bot'] nobody
426-81156
1 year ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-topology t-order 34/14 Mathlib/Topology/Constructions.lean,Mathlib/Topology/Order/LowerUpperTopology.lean 2 13 ['Ruben-VandeVelde', 'TwoFX', 'github-actions', 'jcommelin', 'mans0954', 'mathlib-bors', 'riccardobrasca'] nobody
426-4510
1 year ago
unknown
unknown
16637 astrainfinita
author:astrainfinita
perf: reorder `extends` of `(Add)Monoid` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-algebra
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 ['astrainfinita', 'github-actions', 'leanprover-bot'] nobody
426-3748
1 year ago
unknown
unknown
18765 astrainfinita
author:astrainfinita
chore: changing `outParam` of `MulActionSemiHomClass` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra
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 ['astrainfinita', 'github-actions', 'leanprover-bot'] nobody
425-46409
1 year ago
unknown
unknown
14739 urkud
author:urkud
feat(Measure): add `gcongr` lemmas --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-measure-probability merge-conflict awaiting-author 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
425-3444
1 year ago
unknown
unknown
15822 kmill
author:kmill
feat: greedy colorings of finite graphs Proves that the greedy coloring only takes `G.maxDegree + 1` colors. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-combinatorics 159/0 Mathlib/Combinatorics/SimpleGraph/ConcreteColorings.lean 1 1 ['github-actions'] nobody
422-71602
1 year ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-category-theory 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
422-67130
1 year ago
unknown
unknown
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
422-48773
1 year ago
unknown
unknown
10476 shuxuezhuyi
author:shuxuezhuyi
feat(Topology/UniformSpace): define uniform preordered space We define the semi-uniform structure and the uniform preordered space. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-topology 94/0 Mathlib.lean,Mathlib/Topology/UniformSpace/UniformOrder.lean,docs/references.bib 3 2 ['shuxuezhuyi'] nobody
421-53784
1 year ago
unknown
unknown
17593 astrainfinita
author:astrainfinita
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra blocked-by-other-PR t-order
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 4 ['astrainfinita', 'github-actions', 'mathlib4-dependent-issues-bot', 'vihdzp'] nobody
420-77126
1 year ago
unknown
unknown
17623 astrainfinita
author:astrainfinita
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra awaiting-zulip t-order
label:t-algebra$
146/44 Mathlib/Algebra/Order/GroupWithZero/Canonical.lean,Mathlib/Algebra/Order/GroupWithZero/Unbundled.lean 2 11 ['YaelDillies', 'astrainfinita', 'github-actions', 'j-loreaux'] nobody
420-77126
1 year ago
unknown
unknown
18969 alreadydone
author:alreadydone
chore: generalize Module to NonUnitalSemiring --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-algebra
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
419-14378
1 year ago
unknown
unknown
17624 astrainfinita
author:astrainfinita
feat(Algebra/Order/GroupWithZero/Unbundled): generalize lemmas --- - [ ] depends on: #17623 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra blocked-by-other-PR t-order
label:t-algebra$
121/26 Mathlib/Algebra/Order/GroupWithZero/Unbundled.lean 1 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
417-27898
1 year ago
unknown
unknown
17513 astrainfinita
author:astrainfinita
perf: do not search algebraic hierarchies when using `map_*` lemmas --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-algebra awaiting-bench
label:t-algebra$
5/3 Mathlib/Algebra/Group/Hom/Defs.lean,Mathlib/GroupTheory/GroupAction/Hom.lean 2 10 ['astrainfinita', 'github-actions', 'grunweg', 'leanprover-bot'] nobody
415-73320
1 year ago
unknown
unknown
17515 astrainfinita
author:astrainfinita
perf: do not need `simp low` now --- - [ ] depends on: #17513 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra 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
415-73319
1 year ago
unknown
unknown
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra
label:t-algebra$
25/0 Mathlib.lean,Mathlib/LinearAlgebra/VectorSpace.lean,scripts/noshake.json 3 10 ['Julian', 'PieterCuijpers', 'github-actions', 'urkud'] nobody
414-78565
1 year ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-data 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
412-54642
1 year ago
unknown
unknown
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-topology 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
408-81989
1 year ago
unknown
unknown
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] [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra workshop-AIM-AG-2024 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
405-85647
1 year ago
unknown
unknown
18756 astrainfinita
author:astrainfinita
refactor: deprecate `DistribMulActionSemiHomClass` `MulSemiringActionSemiHomClass` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra
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
401-20311
1 year ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra new-contributor
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
398-32780
1 year ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
396-80106
1 year ago
unknown
unknown
11142 hmonroe
author:hmonroe
feat(ProofTheory): Define logical symbols abstractly; opens new top-level section, drawing from lean4-logic --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-logic 468/1 Mathlib.lean,Mathlib/Data/Fin/VecNotation.lean,Mathlib/ProofTheory/LogicSymbol.lean 3 19 ['PatrickMassot', 'YaelDillies', 'avigad', 'fpvandoorn', 'github-actions'] nobody
391-3526
1 year ago
unknown
unknown
11210 hmonroe
author:hmonroe
Test commit --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
391-3525
1 year ago
unknown
unknown
19621 Command-Master
author:Command-Master
feat: Multiplicity and prime-adic valuation of derivations --- - [ ] depends on: #19596 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra blocked-by-other-PR large-import
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
390-72186
1 year ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-algebra blocked-by-other-PR t-category-theory merge-conflict
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
390-63481
1 year ago
unknown
unknown
18294 astrainfinita
author:astrainfinita
perf: make `Mul.toSMul` higher priority --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-bench t-algebra
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 ['astrainfinita', 'github-actions', 'leanprover-bot'] nobody
385-71118
1 year ago
unknown
unknown
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) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra blocked-by-other-PR t-order merge-conflict awaiting-author
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
377-44415
1 year ago
unknown
unknown
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-order 231/0 Mathlib.lean,Mathlib/Algebra/Order/EFloor.lean,Mathlib/Data/ENat/Basic.lean 3 5 ['YaelDillies', 'github-actions', 'kkytola', 'urkud'] nobody
377-44292
1 year ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP awaiting-author t-meta 82/0 Mathlib.lean,Mathlib/Tactic/DeriveLinearOrder.lean 2 5 ['ChrisHughes24', 'kim-em', 'kmill', 'vihdzp'] nobody
375-18945
1 year ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-meta 517/0 Mathlib.lean,Mathlib/Tactic/DeriveInfinite.lean,test/DeriveInfinite.lean 3 11 ['TimothyGu', 'digama0', 'eric-wieser', 'grunweg', 'kim-em', 'kmill'] kmill
assignee:kmill
375-18944
1 year ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra RFC t-logic
label:t-algebra$
34/13 Mathlib/ModelTheory/Algebra/Ring/Basic.lean 1 10 ['ChrisHughes24', 'YaelDillies', 'awainverse', 'github-actions', 'jcommelin'] nobody
373-36485
1 year ago
unknown
unknown
20459 Ruben-VandeVelde
author:Ruben-VandeVelde
chore: fix names of roots_C_mul_X_{add,sub}_C_of_IsUnit --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-algebra
label:t-algebra$
11/5 Mathlib/Algebra/Polynomial/FieldDivision.lean,Mathlib/Algebra/Polynomial/Roots.lean 2 2 ['eric-wieser', 'github-actions'] nobody
371-60928
1 year ago
unknown
unknown
19462 joelriou
author:joelriou
feat(AlgebraicGeometry): étale sheafification After #19096 and #18945 are merged, if `S : Scheme.{u}`, we shall get instances like `HasSheafify (smallEtaleTopology S) (Type (u + 1))` which means that in order to sheafify preshaves over the small étale site of `S`, we need to assume a certain bump in the universe in the target category. With the main result in this PR (there are still a few sorries), we shall get `HasSheafify (smallEtaleTopology S) (Type u)`. Then, in the subsequent development of étale formalism, we can work in `Type u` (or `Ab.{u}`, etc). --- This is a draft. - [ ] depends on: #19444 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-algebraic-geometry blocked-by-other-PR 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
366-71290
1 year ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-topology 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
366-67517
1 year ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-topology new-contributor 27/0 Mathlib/Topology/Order/DenselyOrdered.lean 1 8 ['github-actions', 'vihdzp'] nobody
364-54792
11 months ago
unknown
unknown
18474 astrainfinita
author:astrainfinita
perf: lower the priority of `*WithOne.to*` instances --- From #7873. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict slow-typeclass-synthesis t-algebra t-data
label:t-algebra$
9/2 Mathlib/Algebra/Polynomial/BigOperators.lean,Mathlib/Data/Int/Cast/Defs.lean,Mathlib/Data/Nat/Cast/Defs.lean 3 7 ['astrainfinita', 'eric-wieser', 'github-actions', 'leanprover-bot'] nobody
364-54547
11 months ago
unknown
unknown
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) please-adopt merge-conflict t-differential-geometry 246/6 Mathlib.lean,Mathlib/Geometry/Manifold/Instances/Sphere.lean,Mathlib/Geometry/Manifold/VectorBundle/Sphere.lean 3 1 ['github-actions'] nobody
364-3081
11 months ago
unknown
unknown
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 merge-conflict awaiting-author t-combinatorics new-contributor 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
363-73878
11 months ago
unknown
unknown
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 merge-conflict blocked-by-other-PR t-combinatorics new-contributor 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
363-73878
11 months ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-computability awaiting-author new-contributor 186/0 Mathlib.lean,Mathlib/Computability/Timed/InsertionSort.lean,Mathlib/Computability/Timed/Merge.lean 3 2 ['github-actions', 'trivial1711'] nobody
363-39797
11 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebraic-geometry blocked-by-other-PR workshop-AIM-AG-2024 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
361-58380
11 months ago
unknown
unknown
8362 urkud
author:urkud
feat(Asymptotics): define `ReflectsGrowth` --- - [x] depends on: #8349 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-analysis 268/0 Mathlib.lean,Mathlib/Analysis/Asymptotics/ReflectsGrowth.lean 2 14 ['YaelDillies', 'fpvandoorn', 'github-actions', 'leanprover-community-mathlib4-bot', 'urkud'] nobody
361-47051
11 months ago
unknown
unknown
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-topology 126/0 Mathlib/Logic/Equiv/PartialEquiv.lean,Mathlib/Topology/PartialHomeomorph.lean 2 4 ['alreadydone', 'github-actions', 'winstonyin'] nobody
361-31647
11 months ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-algebra new-contributor
label:t-algebra$
78/0 Mathlib/Algebra/Group/Defs.lean 1 13 ['github-actions', 'hannahfechtner', 'jcommelin', 'kbuzzard', 'kim-em', 'trivial1711'] nobody
360-977
11 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-algebra new-contributor
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
358-61456
11 months ago
unknown
unknown
19352 hrmacbeth
author:hrmacbeth
chore: change some `nlinarith`s to `linear_combination`s --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
357-4267
11 months ago
unknown
unknown
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`) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-measure-probability new-contributor 203/40 Mathlib/MeasureTheory/Function/LpSeminorm/CompareExp.lean,Mathlib/MeasureTheory/Function/LpSpace.lean 2 1 ['github-actions'] nobody
351-78804
11 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-linter awaiting-author tech debt 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
350-47267
11 months ago
unknown
unknown
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? --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-meta 12/1 Mathlib/Tactic/Linarith/Preprocessing.lean 1 3 ['Vierkantor', 'harahu', 'kim-em', 'mo271'] nobody
349-69397
11 months ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-algebra merge-conflict help-wanted t-topology
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
349-46902
11 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra t-topology 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 2 ['github-actions', 'leanprover-community-mathlib4-bot'] nobody
349-46779
11 months ago
unknown
unknown
21384 alreadydone
author:alreadydone
experiment: make submodule quotient reducibly defeq to additive group quotient --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
1/1 Mathlib/LinearAlgebra/Quotient/Defs.lean 1 1 ['github-actions'] nobody
345-58544
11 months ago
unknown
unknown
9449 hmonroe
author:hmonroe
feat: Add Turing machine with the quintet definition (TMQ) and a chainable step function for each TM type --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-computability awaiting-author 458/1 Mathlib/Computability/TuringMachine.lean,Mathlib/Logic/PartArith.lean 2 8 ['eric-wieser', 'github-actions', 'hmonroe'] nobody
344-11581
11 months ago
unknown
unknown
21496 alreadydone
author:alreadydone
experiment: make SetLike.coe reducible --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data bench-after-CI 1/1 Mathlib/Data/SetLike/Basic.lean 1 1 ['github-actions'] nobody
342-78363
11 months ago
unknown
unknown
18719 astrainfinita
author:astrainfinita
perf: lower the priority of `SemilinearMapClass.toAddHomClass` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict slow-typeclass-synthesis t-algebra awaiting-bench
label:t-algebra$
14/7 Mathlib/Algebra/Module/LinearMap/Defs.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Unique.lean,MathlibTest/TCSynth.lean 3 4 ['astrainfinita', 'github-actions', 'leanprover-bot'] nobody
342-72798
11 months ago
unknown
unknown
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-data 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
341-53999
11 months ago
unknown
unknown
19353 hrmacbeth
author:hrmacbeth
chore: golf some term/rw proofs using `linear_combination` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
340-53120
11 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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR large-import new-contributor merge-conflict awaiting-author t-topology 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
339-36114
11 months ago
unknown
unknown
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
338-72005
11 months ago
unknown
unknown
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
338-72004
11 months ago
unknown
unknown
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
338-72003
11 months ago
unknown
unknown
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-topology 332/0 Mathlib.lean,Mathlib/Topology/UniformSpace/Basic.lean,Mathlib/Topology/UniformSpace/CompletelyRegular.lean 3 6 ['ADedecker', 'adri326'] ADedecker
assignee:ADedecker
338-47531
11 months ago
unknown
unknown
18785 erdOne
author:erdOne
feat(CategoryTheory): command that generates instances for `MorphismProperty` Co-authored-by: Calle Sönne --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-category-theory t-meta 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
336-64041
11 months ago
unknown
unknown
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... [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-linter 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
335-4265
11 months ago
unknown
unknown
16311 madvorak
author:madvorak
feat(Computability): regular languages are context-free --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-computability 72/0 Mathlib.lean,Mathlib/Computability/Chomsky.lean,Mathlib/Computability/ContextFreeGrammar.lean 3 7 ['Rida-Hamadani', 'YaelDillies', 'github-actions', 'madvorak'] nobody
334-70460
11 months ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-computability awaiting-author new-contributor 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
334-70213
11 months ago
unknown
unknown
17005 YnirPaz
author:YnirPaz
feat(SetTheory/Cardinal/Regular): define singular cardinals Define singular cardinals and prove basic lemmas about them. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-set-theory 94/1 Mathlib.lean,Mathlib/SetTheory/Cardinal/Regular.lean,Mathlib/SetTheory/Ordinal/Basic.lean 3 28 ['YaelDillies', 'YnirPaz', 'github-actions', 'vihdzp'] nobody
332-17169
10 months ago
unknown
unknown
18952 Command-Master
author:Command-Master
chore: deprecate `Trunc` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-data 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
331-54786
10 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-algebra new-contributor
label:t-algebra$
43/0 Mathlib/Algebra/BigOperators/Group/Finset/Basic.lean 1 1 ['github-actions', 'j-loreaux'] nobody
329-38984
10 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-meta 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
329-26641
10 months ago
unknown
unknown
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) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict modifies-tactic-syntax awaiting-author t-meta 181/0 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Prune.lean,test/Prune.lean 4 5 ['adomani', 'j-loreaux', 'kmill'] nobody
328-80348
10 months ago
unknown
unknown
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
327-46012
10 months ago
unknown
unknown
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) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author carleson t-measure-probability 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
327-45201
10 months ago
unknown
unknown
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
326-53885
10 months ago
unknown
unknown
20454 urkud
author:urkud
chore(TangentCone): review names Also add some `@[simp]` attrs. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-analysis 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
323-5381
10 months ago
unknown
unknown
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
322-66514
10 months ago
unknown
unknown
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
322-64878
10 months ago
unknown
unknown
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` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-logic 97/43 Mathlib/ModelTheory/LanguageMap.lean,Mathlib/ModelTheory/Order.lean 2 9 ['YaelDillies', 'awainverse', 'github-actions'] nobody
322-44249
10 months ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-data 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
321-43880
10 months ago
unknown
unknown
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) ``` merge-conflict t-algebra t-category-theory new-contributor
label:t-algebra$
47/8 Mathlib/RepresentationTheory/FDRep.lean 1 19 ['github-actions', 'grhkm21', 'joelriou', 'kim-em', 'mathlib-bors'] nobody
320-78811
10 months ago
unknown
unknown
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) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-data 66/0 Mathlib.lean,Mathlib/Data/TypeFun.lean 2 9 ['YaelDillies', 'alexkeizer', 'github-actions', 'leanprover-community-mathlib4-bot'] nobody
319-56842
10 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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict awaiting-author t-topology t-analysis
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
317-79932
10 months ago
unknown
unknown
19372 Command-Master
author:Command-Master
find defeq abuse using diagnostics --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) - [ ] depends on: #19177 merge-conflict blocked-by-other-PR large-import 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
317-79432
10 months ago
unknown
unknown
22408 JLimperg
author:JLimperg
Aesop forward bench: precomp only rpinf --- Not a real PR (yet), just for benchmarking. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict dependency-bump 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
317-68336
10 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR new-contributor t-logic 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
317-21235
10 months ago
unknown
unknown
20636 eric-wieser
author:eric-wieser
feat: multiplication of intervals in rings --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-algebra
label:t-algebra$
36/1 Mathlib/Algebra/Order/Interval/Basic.lean 1 16 ['Timeroot', 'YaelDillies', 'eric-wieser', 'github-actions'] nobody
316-51901
10 months ago
unknown
unknown
16000 YaelDillies
author:YaelDillies
feat: Croot-Sisask Almost Periodicity Almost periodicity is nowadays a standard tool in additive combinatorics. From LeanAPAP --- - [ ] depends on: #15443 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics t-analysis blocked-by-other-PR 0/0 0 4 ['github-actions', 'leanprover-community-mathlib4-bot', 'mergify'] nobody
315-81222
10 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP blocked-by-other-PR t-category-theory large-import merge-conflict 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
315-68483
10 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-topology new-contributor 285/1 Mathlib.lean,Mathlib/Topology/ContinuousMap/MvPolynomial.lean,Mathlib/Topology/ContinuousMap/StoneWeierstrass.lean 3 1 ['github-actions'] nobody
315-64825
10 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP blocked-by-other-PR merge-conflict CI t-meta 66/15 Cache/IO.lean,Cache/Lean.lean,Cache/Requests.lean 3 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
313-83079
10 months ago
unknown
unknown
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) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict large-import 126/0 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter.lean,Mathlib/Tactic/Linter/FindDefEqAbuse.lean,MathlibTest/FindDefEqAbuse.lean 5 1 ['github-actions'] nobody
313-66838
10 months ago
unknown
unknown
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! --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-linter large-import 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
313-65757
10 months ago
unknown
unknown
22648 adomani
author:adomani
test: lean implementation decl diff quandle --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
313-7660
10 months ago
unknown
unknown
18470 astrainfinita
author:astrainfinita
perf: lower the priority of `Normed*.to*` instances --- From #7873. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict slow-typeclass-synthesis t-algebra t-analysis
label:t-algebra$
28/0 Mathlib/Analysis/Normed/Field/Basic.lean,Mathlib/Analysis/Normed/Group/Basic.lean 2 9 ['astrainfinita', 'github-actions', 'jcommelin', 'leanprover-bot'] nobody
311-36252
10 months ago
unknown
unknown
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-differential-geometry 50/0 Mathlib/Geometry/Manifold/Diffeomorph.lean 1 1 ['github-actions'] nobody
310-47733
10 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-set-theory 18/0 Mathlib/SetTheory/Cardinal/Cofinality.lean 1 8 ['YnirPaz', 'github-actions', 'vihdzp'] nobody
310-29128
10 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-topology 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
309-60321
10 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-meta 49/49 Cache/Hashing.lean,Cache/IO.lean,lake-manifest.json 3 8 ['digama0', 'eric-wieser', 'github-actions', 'leanprover-community-mathlib4-bot'] nobody
308-35984
10 months ago
unknown
unknown
22434 qawbecrdtey
author:qawbecrdtey
feat(Mathlib/Analysis/Normed/Lp/WithLp): Added more instances for `WithLp` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-analysis 51/22 Mathlib/Analysis/Normed/Lp/WithLp.lean 1 11 ['eric-wieser', 'github-actions', 'leanprover-bot', 'qawbecrdtey'] nobody
307-65423
10 months ago
unknown
unknown
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`. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-analysis new-contributor 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
307-60651
10 months ago
unknown
unknown
22660 Ruben-VandeVelde
author:Ruben-VandeVelde
chore: follow naming convention around Group.IsNilpotent --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra
label:t-algebra$
133/67 Mathlib/GroupTheory/Frattini.lean,Mathlib/GroupTheory/Nilpotent.lean,Mathlib/GroupTheory/SpecificGroups/ZGroup.lean 3 1 ['github-actions'] nobody
304-680
9 months ago
unknown
unknown
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-linter 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
303-32714
9 months ago
unknown
unknown
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-category-theory infinity-cosmos 22/1 Mathlib/CategoryTheory/Enriched/Limits/HasConicalLimits.lean 1 1 ['github-actions'] nobody
302-85839
9 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-category-theory infinity-cosmos 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
302-38320
9 months ago
unknown
unknown
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`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-algebra
label:t-algebra$
92/16 Mathlib/Algebra/BigOperators/Fin.lean 1 14 ['YaelDillies', 'eric-wieser', 'github-actions', 'quangvdao'] nobody
301-54747
9 months ago
unknown
unknown
20389 eric-wieser
author:eric-wieser
feat: generalize results to `WithLp 0` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-analysis 116/53 Mathlib/Analysis/Normed/Lp/PiLp.lean 1 1 ['github-actions'] nobody
300-43295
9 months ago
unknown
unknown
19189 YnirPaz
author:YnirPaz
feat(SetTheory/Ordinal/Arithmetic): order isomorphism between omega and the natural numbers --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-set-theory 44/0 Mathlib/Order/SuccPred/Limit.lean,Mathlib/SetTheory/Ordinal/Arithmetic.lean 2 21 ['YaelDillies', 'YnirPaz', 'github-actions', 'vihdzp'] nobody
300-24380
9 months ago
unknown
unknown
23142 joneugster
author:joneugster
feat(CategoryTheory/Enriched/Limits): add API for HasConicalLimit --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-category-theory infinity-cosmos 52/9 Mathlib/CategoryTheory/Enriched/Limits/HasConicalLimits.lean 1 2 ['github-actions', 'joelriou'] nobody
300-2585
9 months ago
unknown
unknown
23145 joneugster
author:joneugster
feat(CategoryTheory/Enriched/Limits): add IsConicalLimits --- - [ ] depends on: #23142 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR t-category-theory infinity-cosmos 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
299-55538
9 months ago
unknown
unknown
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) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author CI 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
298-73783
9 months ago
unknown
unknown
20874 grunweg
author:grunweg
chore(nolint.yml): use shallow clones This should be sufficient, and be slightly faster on CI. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author CI 0/3 .github/workflows/nolints.yml 1 2 ['bryangingechen', 'github-actions'] nobody
298-73538
9 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-topology t-order 161/9 Mathlib/Data/ENat/Basic.lean,Mathlib/Topology/Instances/ENat.lean 2 4 ['YaelDillies', 'github-actions', 'leanprover-community-mathlib4-bot'] nobody
294-31315
9 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 α)`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-set-theory t-data 51/0 Mathlib.lean,Mathlib/Data/ENat/Pow.lean 2 1 ['github-actions'] nobody
293-10508
9 months ago
unknown
unknown
16009 Command-Master
author:Command-Master
acyclic graph --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-combinatorics 232/0 Mathlib/Combinatorics/SimpleGraph/Acyclic.lean 1 1 ['github-actions'] nobody
292-65864
9 months ago
unknown
unknown
20613 grunweg
author:grunweg
chore: golf using `List.toArrayMap` --- Depends on batteries#1090 landing in mathlib. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict large-import 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
290-30281
9 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR t-analysis 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
290-1583
9 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict tech debt t-topology RFC 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
289-19887
9 months ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data enhancement new-contributor merge-conflict awaiting-author 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 17 ['chrisflav', 'eric-wieser', 'github-actions', 'j-loreaux', 'markimunro'] nobody
289-9650
9 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 - [ ] [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
288-35480
9 months ago
unknown
unknown
20746 JLimperg
author:JLimperg
Aesop forward branch test --- This is not a real PR; I just want to benchmark this Aesop branch. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
287-79286
9 months ago
unknown
unknown
22810 pechersky
author:pechersky
feat(Counterexamples): metric space not induced by norm Because the distance is not homogeneous --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) - [x] depends on: #22845 merge-conflict WIP t-topology t-analysis 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
287-71942
9 months ago
unknown
unknown
13124 astrainfinita
author:astrainfinita
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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 ['MichaelStollBayreuth', 'astrainfinita', 'github-actions', 'leanprover-bot', 'mathlib4-dependent-issues-bot'] nobody
287-13519
9 months ago
unknown
unknown
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)) ``` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-measure-probability 37/28 Mathlib/MeasureTheory/Decomposition/Exhaustion.lean,Mathlib/MeasureTheory/Measure/Typeclasses.lean 2 4 ['RemyDegenne', 'github-actions', 'sgouezel'] nobody
286-18673
9 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict delegated 8/0 lakefile.lean 1 20 ['YaelDillies', 'adomani', 'eric-wieser', 'github-actions', 'grunweg', 'mathlib-bors'] nobody
285-69241
9 months ago
unknown
unknown
22727 grunweg
author:grunweg
feat: rewrite the isolated by and colon linters in Lean --- - depends on #22726 - depends on: #22728 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-linter 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
284-44959
9 months ago
unknown
unknown
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 t-measure-probability new-contributor merge-conflict awaiting-author t-analysis 60/1 Mathlib/MeasureTheory/Integral/FundThmCalculus.lean 1 3 ['github-actions', 'hrmacbeth', 'victorliu5296'] nobody
284-4639
9 months ago
unknown
unknown
22888 plp127
author:plp127
perf: replace `Lean.Expr.swapBVars` with a better? implementation Replaces `Lean.Expr.swapBVars` with a version that traverses the expression. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-meta 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
282-84084
9 months ago
unknown
unknown
15943 urkud
author:urkud
feat: add `ProdQuotientMapSpace` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-topology 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
282-23011
9 months ago
unknown
unknown
22579 kvanvels
author:kvanvels
doc(Topology/Defs/Induced): fix comments on three functions related to RestrictGenTopology --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-topology documentation awaiting-author 10/9 Mathlib/Topology/Defs/Induced.lean,Mathlib/Topology/RestrictGen.lean 2 4 ['github-actions', 'kvanvels', 'leanprover-community-bot-assistant', 'urkud'] nobody
281-11542
9 months ago
unknown
unknown
19771 robertylewis
author:robertylewis
perf: qqify two functions in linarith --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-meta 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
280-77448
9 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-analysis new-contributor 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
280-76959
9 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-category-theory new-contributor 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
280-73227
9 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-category-theory large-import 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
280-73225
9 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR t-category-theory large-import 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
280-72698
9 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR t-category-theory large-import 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
280-72698
9 months ago
unknown
unknown
13653 adomani
author:adomani
feat: the unusedSetOptionIn linter --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-linter large-import 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
280-17663
9 months ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
279-85759
9 months ago
unknown
unknown
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-topology new-contributor 281/1 Mathlib.lean,Mathlib/Topology/Covering/Basic.lean,Mathlib/Topology/Covering/Lift.lean 3 9 ['alreadydone', 'github-actions', 'grunweg', 'vbeffara'] nobody
279-75955
9 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-category-theory 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
279-9564
9 months ago
unknown
unknown
6252 michaellee94
author:michaellee94
feat(Geometry/Manifolds/Instances/Homeomorph): Homeomorphism maps `C^k` manifolds to `C^k` manifolds --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-differential-geometry 116/0 Mathlib.lean,Mathlib/Geometry/Manifold/Instances/Graph.lean 2 2 ['leanprover-community-bot-assistant', 'michaellee94'] nobody
278-70420
9 months ago
unknown
unknown
24040 astrainfinita
author:astrainfinita
refactor: unbundle algebra from `(NonUnital){Seminormed, Normed}(Comm)Ring` --- - [ ] depends on: #23966 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra blocked-by-other-PR merge-conflict slow-typeclass-synthesis t-analysis
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 5 ['astrainfinita', 'github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
275-66658
9 months ago
unknown
unknown
16314 astrainfinita
author:astrainfinita
chore(Data/Quot): deprecate `ind*'` APIs --- - [x] depends on: #16264 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-data 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
275-11791
9 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) This includes part of #23750 merge-conflict t-data 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
274-81844
8 months ago
unknown
unknown
24060 eric-wieser
author:eric-wieser
chore(MeasureTheory): use `0` instead of `const _ 0` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-measure-probability 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
274-71539
8 months ago
unknown
unknown
24058 astrainfinita
author:astrainfinita
refactor: unbundle algebra from `*NormedField` --- - [ ] depends on: #24040 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra blocked-by-other-PR merge-conflict slow-typeclass-synthesis t-analysis
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 ['astrainfinita', 'github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
274-61449
8 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
274-43444
8 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-category-theory awaiting-CI 22/21 Mathlib/CategoryTheory/EssentialImage.lean,Mathlib/CategoryTheory/Monoidal/Braided.lean,Mathlib/CategoryTheory/Monoidal/Subcategory.lean 3 1 ['grunweg'] nobody
274-43323
8 months ago
unknown
unknown
7874 astrainfinita
author:astrainfinita
chore: make `IsScalarTower A A B` and `IsScalarTower A B B` higher priority --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict slow-typeclass-synthesis t-algebra awaiting-CI
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
274-43298
8 months ago
unknown
unknown
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) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author CI t-meta 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
274-43256
8 months ago
unknown
unknown
5952 eric-wieser
author:eric-wieser
feat: add Qq wrappers for ToExpr --- - [ ] depends on: #6699 (to appease the linter) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-CI t-meta 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
274-43124
8 months ago
unknown
unknown
15483 astrainfinita
author:astrainfinita
chore(GroupTheory/Coset): reduce defeq abuse --- - [x] depends on: #15482 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra
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 ['astrainfinita', 'eric-wieser', 'github-actions', 'grunweg', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'mattrobball', 'mergify', 'urkud'] nobody
274-43084
8 months ago
unknown
unknown
16594 astrainfinita
author:astrainfinita
perf: reorder `extends` and remove some instances in algebra hierarchy --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict slow-typeclass-synthesis t-algebra
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 ['astrainfinita', 'github-actions', 'grunweg', 'leanprover-bot'] nobody
274-42860
8 months ago
unknown
unknown
24106 astrainfinita
author:astrainfinita
refactor: unbundle algebra from `*CStarAlgebra` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) - [ ] depends on: #24058 t-algebra blocked-by-other-PR merge-conflict slow-typeclass-synthesis t-analysis
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 ['astrainfinita', 'github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
274-14590
8 months ago
unknown
unknown
13780 adomani
author:adomani
deprecate injective --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
274-10374
8 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR CI t-meta 231/118 Cache/Hashing.lean,Cache/IO.lean,Cache/Main.lean 3 16 ['github-actions', 'grunweg', 'joneugster', 'kim-em', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
272-53103
8 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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR CI t-meta 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
272-52979
8 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra 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
272-47200
8 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-meta 38/2 Cache/Main.lean 1 11 ['Julian', 'arthurpaulino', 'fpvandoorn', 'github-actions', 'grunweg'] nobody
272-47187
8 months ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-analysis new-contributor 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
272-47153
8 months ago
unknown
unknown
22698 Kiolt
author:Kiolt
feat: notation for whisker(Left/Right)Iso From Toric --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-category-theory toric 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
272-46982
8 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics 14/17 Mathlib/Combinatorics/Optimization/ValuedCSP.lean 1 1 ['github-actions'] nobody
272-46700
8 months ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-algebra new-contributor
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
272-43285
8 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-analysis 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
270-65663
8 months ago
unknown
unknown
12605 astrainfinita
author:astrainfinita
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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 ['YaelDillies', 'astrainfinita', 'eric-wieser', 'github-actions', 'leanprover-community-mathlib4-bot', 'urkud'] nobody
270-60278
8 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-category-theory 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 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
268-3725
8 months ago
unknown
unknown
23859 urkud
author:urkud
feat(Topology/../Order/Field): generalize to `Semifield` .. from a linear ordered field to a linear ordered semifield--- - [ ] depends on: #23857 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-topology 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
267-86101
8 months ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-algebra toric
label:t-algebra$
193/0 Mathlib/LinearAlgebra/LinearIndependent/Tprod.lean 1 1 ['github-actions'] nobody
267-65533
8 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-order 231/89 Mathlib/Order/Interval/Finset/SuccPred.lean,Mathlib/Order/Interval/Set/SuccPred.lean 2 2 ['github-actions', 'leanprover-community-bot-assistant'] nobody
265-62876
8 months ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra
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
265-51573
8 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) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) This is started from the mathport output on https://github.com/leanprover-community/mathlib/pull/19244 merge-conflict t-analysis awaiting-zulip 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
265-32503
8 months ago
unknown
unknown
14931 eric-wieser
author:eric-wieser
feat: volume of a simplex --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-euclidean-geometry 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
263-64030
8 months ago
unknown
unknown
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 . --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-algebra
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
263-61748
8 months ago
unknown
unknown
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) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-analysis 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
262-44886
8 months ago
unknown
unknown
23593 erdOne
author:erdOne
feat(AlgebraicGeometry): the tilde construction is functorial --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-algebraic-geometry 95/38 Mathlib/AlgebraicGeometry/Modules/Sheaf.lean,Mathlib/AlgebraicGeometry/Modules/Tilde.lean 2 4 ['chrisflav', 'github-actions', 'leanprover-community-bot-assistant'] nobody
261-78944
8 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-analysis 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
261-71348
8 months ago
unknown
unknown
22721 grunweg
author:grunweg
chore(MeasureTheory/Function/LpSeminorm/Basic): generalise more results to enorm classes Done for the Carleson project. --- - depends on #22708 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP carleson t-measure-probability 134/10 Mathlib/MeasureTheory/Function/LpSeminorm/Basic.lean 1 2 ['github-actions', 'leanprover-community-bot-assistant'] nobody
260-64016
8 months ago
unknown
unknown
24354 grunweg
author:grunweg
chore(HasFiniteIntegral): rename three lemmas Discovered in #24343. --- - [ ] depends on: #24343 (to avoid merge conflicts) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-measure-probability 108/30 Mathlib/MeasureTheory/Function/L1Space/HasFiniteIntegral.lean 1 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
260-55977
8 months ago
unknown
unknown
23791 SEU-Prime
author:SEU-Prime
Create AmiceTrans.lean --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-number-theory new-contributor 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
260-16897
8 months ago
unknown
unknown
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) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-linter large-import 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
259-69255
8 months ago
unknown
unknown
13649 astrainfinita
author:astrainfinita
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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 ['astrainfinita', 'digama0', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'urkud'] digama0
assignee:digama0
257-35123
8 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-data 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
257-11879
8 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-differential-geometry blocked-by-other-PR 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
257-8068
8 months ago
unknown
unknown
23921 alreadydone
author:alreadydone
Jyxu/projective trace --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-algebra
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
257-7900
8 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-algebra t-category-theory new-contributor
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
257-7724
8 months ago
unknown
unknown
21252 ADedecker
author:ADedecker
feat: redefine uniformly convex normed spaces with filters instead of epsilons And conceptualize some proofs. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-topology t-algebra
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
257-7639
8 months ago
unknown
unknown
19821 eric-wieser
author:eric-wieser
feat: add a Qq version of AtomM that groups by type --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP large-import t-meta 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
257-7452
8 months ago
unknown
unknown
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! --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-core-PR t-meta 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
257-7432
8 months ago
unknown
unknown
17069 yuma-mizuno
author:yuma-mizuno
chore(CategoryTheory/Functor/Basic): put `simp` at `Functor.id_comp` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-category-theory 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
257-7422
8 months ago
unknown
unknown
14803 StevenClontz
author:StevenClontz
chore: use `Disjoint` nhd filters for all separation axioms --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-topology 157/122 Mathlib/Topology/Separation.lean 1 1 ['github-actions'] nobody
257-7406
8 months ago
unknown
unknown
14675 adomani
author:adomani
dev: the repeated variable linter --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-linter 71/0 Mathlib/Tactic/Linter/Lint.lean 1 1 ['github-actions'] nobody
257-7401
8 months ago
unknown
unknown
14330 Ruben-VandeVelde
author:Ruben-VandeVelde
chore: split Mathlib.Algebra.Star.Basic --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
257-7361
8 months ago
unknown
unknown
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! --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-linter 249/0 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter.lean,Mathlib/Tactic/Linter/Papercut.lean,test/Papercut.lean 5 1 ['github-actions'] nobody
257-7246
8 months ago
unknown
unknown
20354 eric-wieser
author:eric-wieser
feat: generalize `ContinuousLinearMap.curry` to TVS Follow on from #10777 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-analysis 57/25 Mathlib/Analysis/NormedSpace/Multilinear/Curry.lean 1 3 ['eric-wieser', 'github-actions', 'leanprover-community-bot-assistant'] nobody
257-7181
8 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-measure-probability 52/46 Mathlib/MeasureTheory/Measure/Haar/Basic.lean 1 0 [] nobody
257-6992
8 months ago
unknown
unknown
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) please-adopt merge-conflict t-algebra
label:t-algebra$
16/4 Mathlib/Algebra/Lie/SkewAdjoint.lean,Mathlib/Algebra/Lie/Subalgebra.lean 2 3 ['eric-wieser', 'ericrbg'] nobody
257-6980
8 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-data 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
257-6974
8 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra
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
257-6969
8 months ago
unknown
unknown
8536 jjaassoonn
author:jjaassoonn
characteristic predicate of tensor product --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra
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
257-6922
8 months ago
unknown
unknown
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`. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-analysis 139/137 Mathlib/Analysis/Distribution/SchwartzSpace.lean,Mathlib/Analysis/Fourier/PoissonSummation.lean,Mathlib/Topology/ContinuousFunction/ZeroAtInfty.lean 3 0 [] nobody
257-6888
8 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP blocked-by-other-PR t-meta 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
257-6884
8 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-algebra
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 2 ['FMLJohn', 'github-actions'] nobody
257-6870
8 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) performance-hack 1/0 lakefile.lean 1 3 ['eric-wieser', 'github-actions', 'leanprover-bot'] nobody
257-6754
8 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`). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-linter 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
257-6721
8 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-linter 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
257-6568
8 months ago
unknown
unknown
14932 eric-wieser
author:eric-wieser
chore: add nndist versions of lemmas --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-analysis 108/1 Mathlib/Analysis/InnerProductSpace/Basic.lean,Mathlib/Geometry/Euclidean/Basic.lean 2 1 ['github-actions'] nobody
257-6534
8 months ago
unknown
unknown
18202 ADedecker
author:ADedecker
chore: refactor algebraic filter bases --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-topology t-algebra
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
255-85605
8 months ago
unknown
unknown
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 ``` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-topology FLT 1/1 Mathlib/Topology/Algebra/UniformMulAction.lean 1 10 ['github-actions', 'leanprover-bot', 'smmercuri', 'urkud'] nobody
255-76938
8 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-euclidean-geometry 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
255-68105
8 months ago
unknown
unknown
15161 adomani
author:adomani
feat(Linter): flag `intros x y` which can be replaced by `intro x y` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-linter 78/1 Mathlib/Tactic/Linter/Lint.lean,test/Lint.lean 2 4 ['adomani', 'github-actions', 'grunweg'] nobody
255-48006
8 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR new-contributor t-computability merge-conflict awaiting-zulip 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
254-40403
8 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-data 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
253-42364
8 months ago
unknown
unknown
19464 adomani
author:adomani
test: removed merge-conflict --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP CI delegated 22/1 .github/workflows/PR_summary.yml,scripts/zulip_emoji_merge_delegate.py 2 10 ['adomani', 'github-actions', 'leanprover-community-bot-assistant'] nobody
252-53688
8 months ago
unknown
unknown
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) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra t-analysis awaiting-CI
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
251-69478
8 months ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author RFC t-data t-meta 27/2 Mathlib/Data/Fin/Tuple/Reflection.lean 1 2 ['github-actions', 'urkud'] nobody
251-38244
8 months ago
unknown
unknown
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) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-differential-geometry blocked-by-other-PR 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
251-37666
8 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-logic 62/0 Mathlib/ModelTheory/Substructures.lean 1 19 ['GabinKolly', 'YaelDillies', 'fpvandoorn', 'github-actions', 'grunweg'] nobody
250-60438
8 months ago
unknown
unknown
24008 meithecatte
author:meithecatte
chore(EpsilonNFA): replace manual lemmas with @[simps] --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-computability awaiting-author new-contributor 2/24 Mathlib/Computability/EpsilonNFA.lean 1 2 ['YaelDillies', 'github-actions', 'urkud'] nobody
248-85982
8 months ago
unknown
unknown
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) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP carleson t-analysis 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
247-62363
8 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict carleson awaiting-CI t-measure-probability 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
246-84047
8 months ago
unknown
unknown
21375 grunweg
author:grunweg
WIP: generalise lemmas to ENorm This work is part of (and a necessary pre-requisite for) the Carleson project. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP awaiting-CI t-measure-probability carleson merge-conflict 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
246-78422
8 months ago
unknown
unknown
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra
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
246-62752
8 months ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-analysis 145/0 Mathlib/Analysis/Convex/Schur.lean 1 16 ['b-mehta', 'eric-wieser', 'github-actions'] nobody
245-73515
8 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order merge-conflict help-wanted awaiting-author t-topology 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
244-74757
7 months ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
243-72659
7 months ago
unknown
unknown
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-linter large-import merge-conflict awaiting-author delegated 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
243-63263
7 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-linter awaiting-author large-import 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
243-63262
7 months ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP awaiting-author t-algebra
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
242-69293
7 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author CI 3/3 .github/build.in.yml,.github/workflows/actionlint.yml 2 12 ['adomani', 'bryangingechen', 'github-actions', 'jcommelin', 'leanprover-community-bot-assistant'] bryangingechen
assignee:bryangingechen
241-14297
7 months ago
unknown
unknown
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`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-category-theory 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 6 ['YaelDillies', 'github-actions', 'leanprover-community-bot-assistant', 'yuma-mizuno'] nobody
237-39868
7 months ago
unknown
unknown
22837 joneugster
author:joneugster
feat(Data/Set/Basic): add subset_iff and not_mem_subset_iff Add `Set.subset_iff` for consistent API with `Finset.subset_iff`. Add `Set.not_mem_subset_iff` and `Finset.not_mem_subset_iff`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-set-theory t-data 9/0 Mathlib/Data/Finset/Defs.lean,Mathlib/Data/Set/Basic.lean 2 4 ['Ruben-VandeVelde', 'github-actions', 'joneugster', 'leanprover-community-bot-assistant'] nobody
234-71105
7 months ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
234-70586
7 months ago
unknown
unknown
24100 eric-wieser
author:eric-wieser
feat: restore some explicit binders from Lean 3 Part of #24099 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author tech debt 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
234-70461
7 months ago
unknown
unknown
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.) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-linter 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
233-76593
7 months ago
unknown
unknown
24163 urkud
author:urkud
refactor(TangentCone): redefine for TVS --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-analysis 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
233-21910
7 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-topology large-import new-contributor 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
232-58323
7 months ago
unknown
unknown
12438 jjaassoonn
author:jjaassoonn
feat: some APIs for flat modules Need horseshoe lemma --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-category-theory 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
227-70949
7 months ago
unknown
unknown
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`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author awaiting-CI t-meta 27/39 Mathlib/Tactic/Recall.lean 1 2 ['github-actions', 'leanprover-community-bot-assistant'] nobody
226-1810
7 months ago
unknown
unknown
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) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-meta 72/5 Mathlib/Util/CountHeartbeats.lean,MathlibTest/CountHeartbeats.lean 2 17 ['adomani', 'github-actions', 'joneugster', 'leanprover-community-bot-assistant', 'mathlib-bors'] adomani
assignee:adomani
226-671
7 months ago
unknown
unknown
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 ``` [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-linter large-import 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 3 ['github-actions', 'grunweg', 'leanprover-community-bot-assistant'] nobody
225-65707
7 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-order 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
224-71432
7 months ago
unknown
unknown
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). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
223-74890
7 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict CI 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
223-21930
7 months ago
unknown
unknown
16062 adomani
author:adomani
Test/ci olean size Tests for oleans --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP awaiting-author CI 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
223-21930
7 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra bench-after-CI
label:t-algebra$
20/35 Mathlib/RingTheory/Valuation/ValuationRing.lean 1 2 ['github-actions', 'leanprover-community-bot-assistant'] nobody
223-13409
7 months ago
unknown
unknown
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`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) please-adopt t-algebra new-contributor merge-conflict awaiting-author
label:t-algebra$
78/0 Mathlib/LinearAlgebra/UnitaryGroup.lean 1 8 ['chrisflav', 'jcommelin', 'leanprover-community-bot-assistant'] nobody
222-30276
7 months ago
unknown
unknown
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`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-data 190/47 Mathlib/Data/Nat/Find.lean 1 2 ['github-actions', 'leanprover-community-bot-assistant'] nobody
221-81965
7 months ago
unknown
unknown
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). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-convex-geometry 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
221-81150
7 months ago
unknown
unknown
23929 meithecatte
author:meithecatte
feat(Computability/NFA): improve bound on pumping lemma --- - [x] depends on: #25321 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-computability awaiting-zulip 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
221-50005
7 months ago
221-50006
221 days ago
0-37135
10 hours
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-topology 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
221-13423
7 months ago
unknown
unknown
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). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP awaiting-author CI 2/1 .github/workflows/PR_summary.yml 1 2 ['github-actions', 'leanprover-community-bot-assistant'] nobody
221-11417
7 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order 33/7 Mathlib/Order/Notation.lean 1 1 ['github-actions'] nobody
220-83113
7 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author delegated t-meta 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
218-30152
7 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict modifies-tactic-syntax t-meta 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
217-35464
7 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author new-contributor t-meta 171/48 Mathlib/Tactic/Polyrith.lean,scripts/polyrith_sage.py 2 16 ['eric-wieser', 'github-actions', 'hanwenzhu', 'kim-em', 'miguelmarco', 'mkoeppe'] nobody
215-22829
7 months ago
unknown
unknown
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
213-66578
6 months ago
unknown
unknown
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 awaiting-author blocked-by-other-PR t-analysis 45/0 Mathlib/Analysis/SpecialFunctions/Trigonometric/Basic.lean 1 3 ['BoltonBailey', 'github-actions', 'mathlib4-dependent-issues-bot'] nobody
213-65291
6 months ago
unknown
unknown
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
213-64722
6 months ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-data 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
212-64309
6 months ago
unknown
unknown
25921 BoltonBailey
author:BoltonBailey
feat: scripts to analyze overlap between namespaces This PR continues the work from #11385. Original PR: https://github.com/leanprover-community/mathlib4/pull/11385 WIP migrated-from-branch t-meta 86/0 scripts/RecordNamespaces.lean,scripts/namespace-overlap.py 2 1 ['github-actions'] nobody
211-52589
6 months ago
211-52605
211 days ago
2-11355
2 days
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-algebra blocked-by-other-PR
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
210-1046
6 months ago
unknown
unknown
18441 ADedecker
author:ADedecker
refactor(AdicTopology): use new API for algebraic filter bases, and factor some code --- - [x] depends on: #18437 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-topology t-algebra
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
209-72891
6 months ago
unknown
unknown
18439 ADedecker
author:ADedecker
refactor: use new algebraic filter bases API in `FiniteAdeleRing` --- - [x] depends on: #18437 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-topology t-algebra
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
209-72889
6 months ago
unknown
unknown
18438 ADedecker
author:ADedecker
refactor: adapt `KrullTopology` to the new algebraic filter bases API --- - [x] depends on: #18437 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-topology t-algebra
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
209-72888
6 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP 18/0 git_hooks/pre-commit 1 1 ['github-actions'] nobody
208-44422
6 months ago
208-44422
208 days ago
0-857
14 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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-data 518/0 Mathlib.lean,Mathlib/Data/DigitExpansion/Defs.lean,docs/references.bib 3 11 ['eric-wieser', 'github-actions', 'kim-em', 'pechersky'] dupuisf
assignee:dupuisf
206-55179
6 months ago
unknown
unknown
21450 eric-wieser
author:eric-wieser
feat: improve trace nodes for `positivity` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta 25/7 Mathlib/Tactic/Positivity/Core.lean 1 1 ['github-actions'] nobody
206-41201
6 months ago
unknown
unknown
26327 eric-wieser
author:eric-wieser
chore: split the tests for positivity --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 528/2 MathlibTest/Positivity/basic.lean,MathlibTest/positivity.lean 2 1 ['github-actions'] nobody
205-39218
6 months ago
unknown
unknown
18662 joelriou
author:joelriou
feat(LinearAlgebra/ExteriorPower): generators of the exterior powers --- - [x] depends on: #18534 - [x] depends on: #18590 - [ ] depends on: #26464 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-algebra blocked-by-other-PR
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
202-7501
6 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-algebra blocked-by-other-PR
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
202-3475
6 months ago
unknown
unknown
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 awaiting-author t-algebra
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
198-3219
6 months ago
unknown
unknown
26581 nomeata
author:nomeata
ignore this: Lean pr testing 9124 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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 0 [] nobody
197-71004
6 months ago
unknown
unknown
15213 adomani
author:adomani
dev: add Mathlib.Tactic.Linter.ForallIntro --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-linter large-import 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
194-22976
6 months ago
unknown
unknown
16074 Rida-Hamadani
author:Rida-Hamadani
feat: combinatorial maps and planar graphs We define combinatorial maps, then we define planar graph using combinatorial maps. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-combinatorics 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
194-20754
6 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-logic 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
194-20753
6 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra awaiting-zulip
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
194-20752
6 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-differential-geometry 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
194-20751
6 months ago
unknown
unknown
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-category-theory 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
194-20628
6 months ago
unknown
unknown
22928 javra
author:javra
feat(CategoryTheory): infrastructure for inclusion morphisms into products in categories with 0-morphisms --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-category-theory 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
194-20246
6 months ago
unknown
unknown
22952 eric-wieser
author:eric-wieser
refactor: reimplement `RingQuot` in terms of `RingCon.Quotient` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra
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
194-20245
6 months ago
unknown
unknown
23763 grunweg
author:grunweg
feat(Linter.openClassical): also lint for Classical declarations as … …a local or scoped instance. --- - [ ] depends on: #23750 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-linter 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
194-20238
6 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-data 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
194-19840
6 months ago
unknown
unknown
24823 eric-wieser
author:eric-wieser
refactor: add `hom` lemmas for the `MonoidalCategory` structure on `ModuleCat` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra
label:t-algebra$
148/164 Mathlib/Algebra/Category/FGModuleCat/Basic.lean,Mathlib/Algebra/Category/ModuleCat/Adjunctions.lean,Mathlib/Algebra/Category/ModuleCat/Monoidal/Basic.lean,Mathlib/Algebra/Category/ModuleCat/Monoidal/Closed.lean,Mathlib/Algebra/Category/ModuleCat/Monoidal/Symmetric.lean,Mathlib/Algebra/Category/ModuleCat/Presheaf/Free.lean,Mathlib/Algebra/Category/ModuleCat/Presheaf/Generator.lean,Mathlib/Algebra/Category/ModuleCat/Presheaf/Monoidal.lean,Mathlib/CategoryTheory/Monoidal/Internal/Module.lean,Mathlib/RepresentationTheory/Coinvariants.lean,Mathlib/RepresentationTheory/Rep.lean 11 21 ['101damnations', 'YaelDillies', 'eric-wieser', 'github-actions', 'joelriou', 'kbuzzard', 'leanprover-community-bot-assistant'] 101damnations
assignee:101damnations
194-19839
6 months ago
194-19839
194 days ago
25-46309
25 days
25071 erdOne
author:erdOne
feat(EllipticCurve): basic API for singular cubics --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebraic-geometry 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
194-19593
6 months ago
unknown
unknown
25197 eric-wieser
author:eric-wieser
feat: Finset.sum induction for tensor products. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra large-import
label:t-algebra$
81/0 Mathlib/LinearAlgebra/TensorProduct/Basic.lean 1 2 ['github-actions', 'leanprover-community-bot-assistant'] nobody
194-19591
6 months ago
unknown
unknown
25218 kckennylau
author:kckennylau
feat(AlgebraicGeometry): Tate normal form of elliptic curves --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebraic-geometry awaiting-zulip new-contributor 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
194-19590
6 months ago
unknown
unknown
25247 alreadydone
author:alreadydone
Projective contraction --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra
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
194-19587
6 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra new-contributor
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
194-19586
6 months ago
unknown
unknown
25561 callesonne
author:callesonne
feat(Category/Grpd): define the bicategory of groupoids --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-category-theory 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
194-19575
6 months ago
210-57298
210 days ago
10-33680
10 days
25671 eric-wieser
author:eric-wieser
refactor: generalize `OreSet` to work for bimodules --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict large-import 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
194-19446
6 months ago
unknown
unknown
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 merge-conflict t-algebraic-geometry 1000/1022 Mathlib/AlgebraicGeometry/EllipticCurve/Jacobian/Basic.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Jacobian/Formula.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Jacobian/Point.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Projective/Basic.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Projective/Formula.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Projective/Point.lean 6 3 ['Multramate', 'github-actions', 'leanprover-community-bot-assistant'] nobody
194-19281
6 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-category-theory 213/0 Mathlib.lean,Mathlib/CategoryTheory/Monoidal/Action/ChosenTypeCopowers.lean 2 2 ['github-actions', 'leanprover-community-bot-assistant'] nobody
194-19279
6 months ago
unknown
unknown
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
194-17291
6 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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-differential-geometry blocked-by-other-PR 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
194-17142
6 months ago
unknown
unknown
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 merge-conflict file-removed t-algebra 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
194-17012
6 months ago
unknown
unknown
26467 joelriou
author:joelriou
feat(LinearAlgebra): the tensor product of a finite family of free modules is free --- - [ ] depends on: #26464 - [ ] depends on: #26465 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-algebra blocked-by-other-PR merge-conflict file-removed
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
194-17010
6 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
193-74675
6 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-topology large-import 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
192-71110
6 months ago
unknown
unknown
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`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-data 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
192-22871
6 months ago
192-42108
192 days ago
3-71177
3 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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 497/0 scripts/DeclarationDiff_text_based.lean 1 4 ['adomani', 'bryangingechen', 'github-actions'] bryangingechen
assignee:bryangingechen
191-2802
6 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-topology 18/0 Mathlib/Topology/StoneCech.lean 1 2 ['github-actions', 'leanprover-community-bot-assistant'] nobody
191-659
6 months ago
191-659
191 days ago
20-8050
20 days
10541 xgenereux
author:xgenereux
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-algebra new-contributor
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', 'YaelDillies', 'eric-wieser', 'fpvandoorn', 'github-actions', 'mariainesdff', 'mathlib4-dependent-issues-bot', 'mattrobball', 'xgenereux'] AntoineChambert-Loir
assignee:AntoineChambert-Loir
189-75068
6 months ago
unknown
unknown
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 merge-conflict t-topology 920/0 Mathlib.lean,Mathlib/Topology/Compactification/OnePointHomeomorph.lean,Mathlib/Topology/Compactification/OnePointRealLemmas.lean 3 3 ['bjoernkjoshanssen', 'github-actions', 'leanprover-community-bot-assistant'] nobody
189-6733
6 months ago
unknown
unknown
26994 Paul-Lez
author:Paul-Lez
feat(Topology/MetricSpace/Pseudo/Defs): add easy lemma about opens in topological spaces Split from #26992 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-topology easy 9/0 Mathlib/Topology/MetricSpace/Pseudo/Defs.lean 1 4 ['Paul-Lez', 'github-actions', 'grunweg'] nobody
187-67859
6 months ago
187-69281
187 days ago
0-8390
2 hours
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-analysis 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
187-58554
6 months ago
unknown
unknown
21039 eric-wieser
author:eric-wieser
hack: override `instance` to insert `fast_instance%` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) please-adopt merge-conflict t-meta 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
187-49761
6 months ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
187-28466
6 months ago
187-69465
187 days ago
2-48079
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author CI t-meta 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
185-50618
6 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-topology new-contributor 63/0 Mathlib/Topology/MetricSpace/HausdorffDimension.lean 1 10 ['AntoineChambert-Loir', 'FrankieNC', 'github-actions', 'grunweg'] nobody
185-48292
6 months ago
185-62703
185 days ago
0-12255
3 hours
25611 erdOne
author:erdOne
chore(RingTheory): add `Algebra (FractionRing R) (FractionRing S)` Co-authored-by: Yakov Pechersky --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra
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
183-75877
5 months ago
217-71563
217 days ago
2-23633
2 days
18230 digama0
author:digama0
feat(Tactic/ScopedNS): extend `scoped[NS]` to more commands refactor `ScopedNS` to remove error prone repetitiveness and extend it to other commands such as `syntax`, `macro`, `elab`, etc. Co-authored-by: Jon Eugster --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-meta 201/26 Mathlib/Tactic/ScopedNS.lean,MathlibTest/scopedNS.lean 2 7 ['adomani', 'digama0', 'eric-wieser', 'github-actions', 'joneugster', 'kbuzzard'] nobody
181-82338
5 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-linter 66/0 Mathlib/Tactic/Linter/TruncatedNat.lean 1 2 ['BoltonBailey', 'eric-wieser', 'github-actions'] nobody
177-26463
5 months ago
unknown
unknown
25284 alreadydone
author:alreadydone
feat(LinearAlgebra/Contraction): bijectivity of `dualTensorHom` + generalize to CommSemiring --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-algebra
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
176-40417
5 months ago
183-6184
183 days ago
10-18736
10 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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-category-theory 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
175-83703
5 months ago
unknown
unknown
26784 eric-wieser
author:eric-wieser
chore: remove suppress_compilation Still not exhaustive. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
175-55964
5 months ago
unknown
unknown
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. merge-conflict WIP t-data 40/0 Mathlib/Data/Sign.lean 1 10 ['eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'madvorak'] nobody
174-86315
5 months ago
unknown
unknown
26987 joelriou
author:joelriou
chore: deprecating module LinearAlgebra.PiTensorProduct --- - [ ] depends on: #26464 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-algebra blocked-by-other-PR
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
174-84716
5 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-analysis 311/0 Mathlib/Analysis/Normed/Algebra/Logarithm.lean 1 1 ['github-actions'] nobody
174-63571
5 months ago
unknown
unknown
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra 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
173-27885
5 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-meta 139/0 Refactor/Main.lean,lakefile.lean 2 11 ['adomani', 'digama0', 'eric-wieser', 'github-actions', 'joneugster', 'leanprover-community-bot-assistant', 'mattrobball'] nobody
169-67876
5 months ago
unknown
unknown
12181 adomani
author:adomani
lint also `let` vs `have` This PR is symmetrical to #12157: here we lint for non-`Type`-valued `let`s. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-linter 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
167-78192
5 months ago
unknown
unknown
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` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebraic-topology WIP t-category-theory new-contributor merge-conflict 720/0 Mathlib.lean,Mathlib/AlgebraicTopology/AugmentedSimplexCategory.lean,Mathlib/AlgebraicTopology/SimplicialObject.lean,Mathlib/Order/Category/FinLinOrd.lean 4 5 ['TwoFX', 'YaelDillies', 'joelriou', 'jstoobysmith'] nobody
167-78130
5 months ago
unknown
unknown
10084 alreadydone
author:alreadydone
draft for Van Kampen The part about the homotopy lifting property for covering maps has been extracted to #22649 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-algebraic-topology 91/24 Mathlib/AlgebraicTopology/FundamentalGroupoid/Basic.lean,Mathlib/AlgebraicTopology/FundamentalGroupoid/VanKampen.lean 2 1 ['leanprover-community-bot-assistant'] nobody
167-78039
5 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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebraic-topology infinity-cosmos t-meta 525/33 Mathlib.lean,Mathlib/AlgebraicTopology/SimplexCategory/Basic.lean,Mathlib/AlgebraicTopology/SimplexCategory/Defs.lean,Mathlib/AlgebraicTopology/SimplicialObject/Basic.lean,Mathlib/Tactic.lean,Mathlib/Tactic/SimplexCategory.lean,Mathlib/Util/Superscript.lean,MathlibTest/SimplexCategory.lean,MathlibTest/SimplicialObject.lean,MathlibTest/superscript.lean,scripts/noshake.json 11 23 ['eric-wieser', 'gio256', 'github-actions', 'kim-em', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] eric-wieser
assignee:eric-wieser
167-77936
5 months ago
unknown
unknown
25914 eric-wieser
author:eric-wieser
feat: add an ext lemma for the opposite category This powers up `aesop_cat`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-category-theory awaiting-CI 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
167-75773
5 months ago
unknown
unknown
27704 vihdzp
author:vihdzp
feat: link `Minimal` and `IsLeast` together --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-order 24/0 Mathlib/Order/Bounds/Basic.lean 1 3 ['b-mehta', 'github-actions'] nobody
167-75217
5 months ago
unknown
unknown
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` [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-algebra
label:t-algebra$
248/0 Mathlib.lean,Mathlib/RingTheory/FractionalIdeal/LocalizedAtPrime.lean 2 2 ['github-actions', 'leanprover-community-bot-assistant'] nobody
167-61016
5 months ago
unknown
unknown
24260 plp127
author:plp127
feat(Topology): add API for Hereditarily Lindelof spaces Copies the stuff about Lindelof spaces to Hereditarily Lindelof spaces. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-topology 222/42 Mathlib/Topology/Compactness/Lindelof.lean 1 15 ['github-actions', 'grunweg', 'mathlib4-merge-conflict-bot', 'urkud'] urkud
assignee:urkud
167-30588
5 months ago
unknown
unknown
27181 ADedecker
author:ADedecker
chore: more conceptual definition of `ValuativeRel.ValueGroupWithZero` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra large-import
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
167-30577
5 months ago
unknown
unknown
27813 javra
author:javra
feat: IMO 2025 Q1 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) IMO WIP 882/0 Archive/Imo/Imo2025Q1.lean 1 1 ['github-actions'] nobody
166-78998
5 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-measure-probability 97/17 Mathlib.lean,Mathlib/MeasureTheory/Measure/Typeclasses/FiniteMoments.lean,Mathlib/Probability/Moments/CovarianceBilin.lean 3 2 ['github-actions', 'mathlib4-merge-conflict-bot'] nobody
166-65453
5 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-number-theory blocked-by-other-PR merge-conflict awaiting-author t-analysis 937/0 Mathlib/NumberTheory/SelbergSieve/Basic.lean,Mathlib/NumberTheory/SelbergSieve/Selberg.lean,docs/references.bib 3 3 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
166-63298
5 months ago
unknown
unknown
27826 xgenereux
author:xgenereux
feat(Subsemiring): mk_eq_zero Add a `mk_eq_zero` lemma for `Subsemiring`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-algebra
label:t-algebra$
4/0 Mathlib/Algebra/Ring/Subsemiring/Defs.lean 1 3 ['eric-wieser', 'github-actions', 'xgenereux'] nobody
166-60480
5 months ago
166-63562
166 days ago
0-6967
1 hour
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-data 183/0 Mathlib/Control/Monad/Cont.lean 1 8 ['BoltonBailey', 'eric-wieser', 'github-actions'] nobody
166-23008
5 months ago
185-40691
185 days ago
0-82325
22 hours
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-meta 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
165-26499
5 months ago
165-73399
165 days ago
15-49725
15 days
26383 eric-wieser
author:eric-wieser
feat: `Real.sin_eq_one_iff` and similar --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-analysis 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
163-84681
5 months ago
unknown
unknown
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 merge-conflict t-algebraic-geometry 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 2 ['github-actions', 'leanprover-community-bot-assistant'] nobody
163-84563
5 months ago
unknown
unknown
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
163-84556
5 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 merge-conflict t-algebraic-geometry 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
163-84551
5 months ago
unknown
unknown
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 merge-conflict t-algebraic-geometry 159/52 Mathlib/AlgebraicGeometry/EllipticCurve/Affine.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Group.lean 2 1 ['Multramate'] nobody
163-84547
5 months ago
unknown
unknown
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 merge-conflict t-algebraic-geometry 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
163-84542
5 months ago
unknown
unknown
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 merge-conflict t-algebraic-geometry 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
163-84537
5 months ago
unknown
unknown
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 merge-conflict t-group-theory 81/12 Mathlib/GroupTheory/GroupAction/Basic.lean,Mathlib/GroupTheory/Subgroup/Basic.lean,Mathlib/GroupTheory/Submonoid/Operations.lean 3 0 [] nobody
163-84531
5 months ago
unknown
unknown
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 merge-conflict t-group-theory 29/6 Mathlib/GroupTheory/Subgroup/Basic.lean,Mathlib/GroupTheory/Submonoid/Operations.lean 2 0 [] nobody
163-84526
5 months ago
unknown
unknown
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` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) - [ ] depends on: #25483 - [ ] depends on: #25485 merge-conflict t-set-theory blocked-by-other-PR new-contributor 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
163-84355
5 months ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) - [ ] depend on: #25483 merge-conflict t-set-theory new-contributor 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
163-84351
5 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) - [ ] depends on: #25483 merge-conflict t-set-theory blocked-by-other-PR new-contributor 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
163-84346
5 months ago
unknown
unknown
25474 adomani
author:adomani
test for .lean/.md check A test PR for #25473. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-linter file-removed 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
163-84340
5 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR t-analysis 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
163-84336
5 months ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra
label:t-algebra$
105/0 Mathlib.lean,Mathlib/LinearAlgebra/Basis/HasCanonicalBasis.lean 2 2 ['github-actions', 'leanprover-community-bot-assistant'] nobody
163-84331
5 months ago
unknown
unknown
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) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) please-adopt merge-conflict t-linter large-import 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
163-84326
5 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-meta new-contributor 17/5 Mathlib/Tactic/ComputeDegree.lean,MathlibTest/ComputeDegree.lean 2 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
163-84321
5 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP IMO large-import 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
163-84281
5 months ago
unknown
unknown
27643 ADedecker
author:ADedecker
Ad bdd unif conv --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
163-63040
5 months ago
unknown
unknown
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 merge-conflict WIP t-ring-theory 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
163-348
5 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-ring-theory 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
163-63
5 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-ring-theory 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
163-15
5 months ago
unknown
unknown
22898 AntoineChambert-Loir
author:AntoineChambert-Loir
feat(RingTheory/TensorProduct/DirectLimit/FG): direct limit of finitely generated submodules and tensor product --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-ring-theory 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
163-8
5 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-ring-theory 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
162-86371
5 months ago
unknown
unknown
20431 erdOne
author:erdOne
feat(RingTheory/AdicCompletion): monotonicity of adic-completeness --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-ring-theory 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
162-86364
5 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-ring-theory large-import 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
162-86349
5 months ago
unknown
unknown
18646 jxjwan
author:jxjwan
feat(RingTheory): isotypic components --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-ring-theory new-contributor 308/0 Mathlib/Order/CompactlyGenerated/Basic.lean,Mathlib/RingTheory/Isotypic.lean,Mathlib/RingTheory/SimpleModule.lean 3 1 ['github-actions'] nobody
162-86342
5 months ago
unknown
unknown
17246 pechersky
author:pechersky
feat(RingTheory/PrimaryDecomposition): PIR of Noetherian under jacobson condition --- - [x] depends on: #17634 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-ring-theory 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
162-86336
5 months ago
unknown
unknown
21474 erdOne
author:erdOne
feat(RingTheory): replace `Ring.DimensionLEOne` with `Ring.KrullDimLE` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-ring-theory large-import 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
162-86280
5 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-ring-theory 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
162-86243
5 months ago
unknown
unknown
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`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-group-theory 206/2 Mathlib/GroupTheory/PresentedGroup.lean,Mathlib/GroupTheory/SpecificGroups/Dihedral.lean 2 6 ['kbuzzard', 'newell'] nobody
162-86079
5 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-group-theory large-import 53/1 Mathlib/GroupTheory/GroupAction/Quotient.lean,Mathlib/Topology/MetricSpace/IsometricSMul.lean 2 6 ['YaelDillies', 'github-actions', 'grunweg', 'urkud'] eric-wieser
assignee:eric-wieser
162-86072
5 months ago
unknown
unknown
27886 alreadydone
author:alreadydone
feat(Algebra): (Mv)Polynomial.X is irreducible assuming NoZeroDivisors --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-algebra
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
162-83807
5 months ago
164-4148
164 days ago
0-70082
19 hours
26200 adomani
author:adomani
fix: add label when landrun fails Adds the `permission-denied` label on PRs that get blocked by landrun. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict CI 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
162-35274
5 months ago
162-35274
162 days ago
46-51722
46 days
17469 joelriou
author:joelriou
feat(Algebra/ModuleCat/Differentials/Presheaf): the presheaf of relative differentials Given a functor `F : C ⥤ D`, presheaves of commutative rings `S`, `R` and a morphism `φ : S ⟶ F.op ⋙ R`, we show that derivations relative to `φ` are representable by a presheaf of `R`-modules. This is obtained by reducing to the case of absolute differentials. The construction shall allow to deduce the presheaf version of the cokernel sequence $$f^\star \Omega_{Y/S} ⟶ \Omega_{X/S} ⟶ \Omega_{X/Y} ⟶ 0$$ when `f : X ⟶ Y` and `g : Y ⟶ S` are morphisms of schemes. --- - [x] depends on: #17366 - [x] depends on: #19507 - [x] depends on: #17388 - [x] depends on: #16755 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-category-theory large-import merge-conflict t-algebraic-geometry 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
162-30623
5 months ago
unknown
unknown
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`.) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-category-theory 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
162-19982
5 months ago
unknown
unknown
27709 kckennylau
author:kckennylau
chore: fix links --- See https://github.com/leanprover-community/mathlib4/pull/27545#discussion_r2238206933 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
162-18193
5 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-algebra
label:t-algebra$
17/0 Mathlib/Algebra/Module/Zlattice.lean 1 3 ['alreadydone', 'newell'] nobody
161-36081
5 months ago
unknown
unknown
27286 edegeltje
author:edegeltje
refactor(OrderDual): make a one-field structure and remove defeq abuse --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-order 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
161-35803
5 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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-data easy 11/9 Mathlib/Algebra/BigOperators/Finsupp/Basic.lean,Mathlib/Data/Finsupp/Indicator.lean 2 3 ['github-actions', 'ocfnash', 'tristan-f-r'] nobody
159-44906
5 months ago
160-2325
160 days ago
0-28703
7 hours
28168 astrainfinita
author:astrainfinita
feat: hensel's lemma for topological rings --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra WIP t-ring-theory t-topology
label:t-algebra$
616/0 Mathlib/RingTheory/Polynomial/Hensel.lean 1 1 ['github-actions'] nobody
158-30341
5 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-number-theory new-contributor large-import 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
158-3483
5 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP awaiting-author t-category-theory 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
157-82850
5 months ago
unknown
unknown
27451 kckennylau
author:kckennylau
feat(RingTheory/Valuation): define ball, closed ball, and sphere *From the 2025 Local Class Field Theory Workshop.* --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-ring-theory 27/0 Mathlib/RingTheory/Valuation/Basic.lean 1 13 ['JovanGerb', 'github-actions', 'kckennylau', 'mathlib4-merge-conflict-bot', 'pechersky', 'wwylele'] nobody
156-67777
5 months ago
156-67778
156 days ago
17-51735
17 days
27987 kckennylau
author:kckennylau
feat(RingTheory/Valuation): define ball, closed ball, and sphere --- The pullback PR of #26827 and #27451. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-ring-theory large-import 73/0 Mathlib/RingTheory/Valuation/Basic.lean 1 4 ['JovanGerb', 'github-actions', 'kckennylau', 'mathlib4-merge-conflict-bot'] nobody
156-67406
5 months ago
156-67407
156 days ago
6-5823
6 days
27444 grunweg
author:grunweg
feat: generalise more lemmas to enorms The selection of lemmas may seem eclectic, but follows a clear path: I'm working on generalising the last section of `IntegrableOn.lean` to enorms. (This will be continued in a later PR.) --- Commits can be reviewed independently. - [x] depends on: #27419 (first commits) - [x] depends on: #27456 (last commits) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
156-63402
5 months ago
unknown
unknown
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) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP carleson t-measure-probability 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
156-61127
5 months ago
unknown
unknown
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 awaiting-author t-combinatorics new-contributor 14/0 Mathlib/Combinatorics/SimpleGraph/Subgraph.lean 1 3 ['b-mehta', 'github-actions', 'xcloudyunx'] b-mehta
assignee:b-mehta
156-19229
5 months ago
156-33309
156 days ago
25-82865
25 days
25133 erdOne
author:erdOne
feat(Tactic/NormNum): support positive characteristic Co-authored-by: Heather Macbeth --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP large-import t-meta 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
154-82566
5 months ago
unknown
unknown
27003 eric-wieser
author:eric-wieser
chore: use `Simp.ResultQ` more often Also uses `~q` in place of manual `isDefEq` matching. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-meta 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
154-82030
5 months ago
154-82031
154 days ago
32-67299
32 days
22925 ggranberry
author:ggranberry
feat(Mathlib/PlaceHolder/ToeplitzHausdorff): Toeplitz-Hausdorff --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP new-contributor will-close-soon awaiting-author help-wanted t-analysis 411/0 Mathlib/PlaceHolder/ToeplitzHausdorff.lean,Mathlib/PlaceHolder/ToeplitzHausdorff_v2.lean 2 11 ['faenuccio', 'ggranberry', 'github-actions'] faenuccio
assignee:faenuccio
154-81753
5 months ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-data new-contributor 103/0 Mathlib/Data/Set/Prod.lean,Mathlib/SetTheory/ZFC/Basic.lean 2 10 ['Ruben-VandeVelde', 'VTrelat', 'github-actions', 'leanprover-community-bot-assistant'] nobody
154-71673
5 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-dynamics t-measure-probability 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
154-50002
5 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-meta 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
154-36826
5 months ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-differential-geometry 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
154-36387
5 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-linter blocked-by-other-PR awaiting-CI 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
154-12321
5 months ago
unknown
unknown
27996 grunweg
author:grunweg
feat: check indentation in doc-strings, medium version --- - [ ] depends on: #27898 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP blocked-by-other-PR 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
154-12196
5 months ago
unknown
unknown
27759 plp127
author:plp127
chore(FreeAbelianGroup): deprecate multiplication Deprecate multiplication on `FreeAbelianGroup` in favor of using `MonoidAlgebra`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra large-import
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
153-3272
5 months ago
unknown
unknown
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. --- please-adopt new-contributor merge-conflict modifies-tactic-syntax good first issue t-meta 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
153-741
5 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict slow-typeclass-synthesis t-algebra 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
152-60176
4 months ago
unknown
unknown
21776 alreadydone
author:alreadydone
Invertible modules --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra
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
152-2821
4 months ago
unknown
unknown
20722 ctchou
author:ctchou
feat(Counterexamples): the Vitali set is non-measurable --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) please-adopt t-measure-probability new-contributor merge-conflict 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
151-79567
4 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP carleson 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
151-71081
4 months ago
unknown
unknown
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
150-3995
4 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-meta 16/0 Mathlib/Control/Monad/Cont.lean 1 25 ['Vierkantor', 'YaelDillies', 'eric-wieser', 'github-actions', 'kmill'] nobody
149-80381
4 months ago
unknown
unknown
28276 eric-wieser
author:eric-wieser
refactor: tidy `lift_unique` lemmas --- - [ ] depends on: #28275 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
149-79652
4 months ago
unknown
unknown
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 blocked-by-other-PR new-contributor merge-conflict awaiting-author t-logic 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
149-14979
4 months ago
152-508
152 days ago
0-32456
9 hours
28631 faenuccio
author:faenuccio
feat(Data\Nat\ModEq.lean): add grind attribute to ModEq --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-data 7/0 Mathlib/Data/Nat/ModEq.lean 1 4 ['faenuccio', 'github-actions', 'leanprover-bot'] nobody
148-86034
4 months ago
unknown
unknown
28622 alreadydone
author:alreadydone
chore(Mathlib): replace `=>` by `↦` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
148-40306
4 months ago
148-40307
148 days ago
0-55389
15 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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-algebra
label:t-algebra$
7/0 Mathlib/LinearAlgebra/UnitaryGroup.lean 1 4 ['github-actions', 'j-loreaux', 'mathlib4-merge-conflict-bot', 'tristan-f-r'] nobody
148-35945
4 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict file-removed blocked-by-other-PR t-category-theory 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
148-13512
4 months ago
unknown
unknown
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". --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-ring-theory 133/0 Mathlib/RingTheory/PowerSeries/Substitution.lean 1 9 ['chrisflav', 'erdOne', 'github-actions', 'kckennylau'] kbuzzard
assignee:kbuzzard
148-5157
4 months ago
148-5157
148 days ago
48-28828
48 days
28680 vihdzp
author:vihdzp
feat: set has cardinality one iff singleton --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-set-theory easy 11/1 Mathlib/SetTheory/Cardinal/Basic.lean,Mathlib/SetTheory/Cardinal/Defs.lean 2 5 ['b-mehta', 'github-actions', 'kckennylau'] nobody
147-71918
4 months ago
147-71918
147 days ago
0-20531
5 hours
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-set-theory 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
147-54117
4 months ago
unknown
unknown
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`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict delegated large-import 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
147-16487
4 months ago
unknown
unknown
28626 alreadydone
author:alreadydone
chore(Archive, Counterexamples): replace => by ↦ --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
146-69432
4 months ago
146-69433
146 days ago
2-46227
2 days
26078 kckennylau
author:kckennylau
feat(AlgebraicGeometry): add x, y, px, py for points on elliptic curves --- Split from #25218. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-algebraic-geometry 44/0 Mathlib/AlgebraicGeometry/EllipticCurve/Affine/Point.lean 1 12 ['MichaelStollBayreuth', 'Multramate', 'acmepjz', 'dagurtomas', 'github-actions', 'kckennylau'] dagurtomas
assignee:dagurtomas
146-66442
4 months ago
146-66442
146 days ago
64-10273
64 days
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra blocked-by-other-PR new-contributor
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
146-51487
4 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author help-wanted t-euclidean-geometry 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
146-28118
4 months ago
unknown
unknown
13795 astrainfinita
author:astrainfinita
perf(Algebra/{Group, GroupWithZero, Ring}/InjSurj): reduce everything --- - [ ] depends on: #15192 - [ ] depends on: #15476 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra
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
145-75503
4 months ago
unknown
unknown
28095 Equilibris
author:Equilibris
Univ generic corec Draft PR: Adding variable universe corecursor for PFunctor --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict new-contributor 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
145-36749
4 months ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-data new-contributor 24/26 Mathlib/Data/TypeVec.lean 1 7 ['Equilibris', 'alexkeizer', 'github-actions', 'mathlib4-merge-conflict-bot'] nobody
145-36748
4 months ago
145-36749
145 days ago
13-47613
13 days
27868 grunweg
author:grunweg
linter indentation playground --- Trying out the changes in #27525. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-linter 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
145-19942
4 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) - [ ] depends on: #25483 - [ ] depends on: #25485 - [ ] depends on: #25486 merge-conflict t-set-theory blocked-by-other-PR new-contributor 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
145-16105
4 months ago
unknown
unknown
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) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict new-contributor 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
145-16068
4 months ago
167-78390
167 days ago
7-51497
7 days
28042 kckennylau
author:kckennylau
feat(Topology/ValuativeRel): a topological basis indexed by pairs of elements --- The pullback PR of #27314 and #27163. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-ring-theory 140/23 Mathlib/RingTheory/Valuation/ValuativeRel.lean,Mathlib/Topology/Algebra/Valued/ValuativeRel.lean 2 3 ['github-actions', 'grunweg', 'mathlib4-merge-conflict-bot'] nobody
145-16022
4 months ago
154-67466
154 days ago
7-2766
7 days
23966 astrainfinita
author:astrainfinita
refactor: unbundle algebra from `{Seminormed, Normed}(Add)(Comm)Group` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) - [ ] depends on: #23621 - [ ] depends on: #23961 t-algebra blocked-by-other-PR merge-conflict slow-typeclass-synthesis t-analysis
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
144-77689
4 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict new-contributor 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
144-64300
4 months ago
167-78391
167 days ago
7-53541
7 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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-data new-contributor 326/0 Mathlib/Data/Nat/Choose/AbelBinomial.lean 1 28 ['ElifUskuplu', 'FrankieNC', 'github-actions', 'iu-isgood'] nobody
144-64061
4 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) please-adopt t-linter RFC 15/0 MathlibTest/DeprecatedSyntaxLinter.lean,MathlibTest/Monotonicity.lean 2 3 ['github-actions', 'grunweg', 'mathlib4-dependent-issues-bot'] nobody
144-63706
4 months ago
unknown
unknown
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict large-import migrated-from-branch t-meta 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
143-68136
4 months ago
154-35893
154 days ago
11-81029
11 days
28787 alreadydone
author:alreadydone
feat(Counterexamples): a domain whose ring of differences is not a domain Example produced by Gemini 2.5 Pro: https://gemini.google.com/share/9558539e1309 --- - [ ] depends on: #28468 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra blocked-by-other-PR large-import
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
143-67511
4 months ago
143-72955
143 days ago
1-9551
1 day
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 awaiting-author t-algebra
label:t-algebra$
10/0 Mathlib/LinearAlgebra/Matrix/NonsingularInverse.lean 1 16 ['eric-wieser', 'github-actions', 'madvorak', 'ocfnash'] nobody
142-2598
4 months ago
unknown
unknown
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.* --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-ring-theory 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
140-66881
4 months ago
160-31492
160 days ago
14-24576
14 days
27785 staroperator
author:staroperator
chore(Algebra/Group/Submonoid): golf `Nat.addSubmonoidClosure_one` using `simp` This should improve the proof readability. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra large-import
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
140-21363
4 months ago
140-21364
140 days ago
26-29321
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] ``` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-meta 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
140-21234
4 months ago
140-21235
140 days ago
12-66568
12 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`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-CI t-measure-probability 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
140-13830
4 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP blocked-by-other-PR t-combinatorics 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
139-71074
4 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP blocked-by-other-PR t-combinatorics 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
139-71073
4 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP blocked-by-other-PR t-combinatorics 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
139-71072
4 months ago
unknown
unknown
26952 robin-carlier
author:robin-carlier
feat(CategoryTheory/DayConvolution): monoid objects internal to day convolutions In this file, given `F : C ⊛⥤ V`, we provide a bijective correspondence between lax monoidal structures on `F.functor` and `Mon_Class F` structures. We also prove that through this correspondance, monoidal natural transformations correspond to morphisms of internal monoid objects. --- - [ ] depends on: #26890 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR t-category-theory 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
139-43283
4 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR t-category-theory 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 6 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
139-43158
4 months ago
184-69612
184 days ago
0-379
6 minutes
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR t-category-theory 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 5 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
139-43156
4 months ago
184-3705
184 days ago
0-474
7 minutes
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR t-category-theory 1585/24 Mathlib.lean,Mathlib/CategoryTheory/Functor/KanExtension/Basic.lean,Mathlib/CategoryTheory/Monoidal/DayConvolution.lean,Mathlib/CategoryTheory/Monoidal/DayConvolution/DayFunctor.lean 4 5 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
139-43155
4 months ago
unknown
unknown
26097 adomani
author:adomani
dev: the relative linter --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP awaiting-author t-linter 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
139-19930
4 months ago
unknown
unknown
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data new-contributor 16/21 Mathlib/Data/PFunctor/Multivariate/W.lean 1 8 ['Equilibris', 'alexkeizer', 'github-actions'] nobody
136-49270
4 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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR new-contributor merge-conflict awaiting-author t-analysis 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
136-47890
4 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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 blocked-by-other-PR t-category-theory large-import merge-conflict 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
135-83350
4 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-category-theory infinity-cosmos 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
135-82740
4 months ago
170-587
170 days ago
15-46601
15 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 merge-conflict t-number-theory blocked-by-other-PR t-analysis 407/83 Mathlib/NumberTheory/Divisors.lean,Mathlib/NumberTheory/SelbergSieve.lean 2 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
135-50000
4 months ago
165-33679
165 days ago
1-36832
1 day
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-linter 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
135-49999
4 months ago
unknown
unknown
25208 erdOne
author:erdOne
feat(LinearAlgebra): `tensor_induction` macro --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-algebra RFC
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
135-17707
4 months ago
unknown
unknown
28017 eric-wieser
author:eric-wieser
feat: generalize some opnorm lemmas to seminormed spaces --- - [ ] depends on: #28014 - [ ] depends on: #28101 - [ ] depends on: #29120 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP blocked-by-other-PR t-analysis 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
134-35482
4 months ago
unknown
unknown
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 t-algebra merge-conflict slow-typeclass-synthesis awaiting-zulip t-analysis
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
134-35235
4 months ago
142-72789
142 days ago
0-16864
4 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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-set-theory 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
134-20923
4 months ago
187-51524
187 days ago
9-66014
9 days
29232 vihdzp
author:vihdzp
feat: more theorems on `SuccAddOrder` We make use of the (relatively) new `CanonicallyOrderedAdd` typeclass in order to generalize various theorems on `Ordinal` to `SuccAddOrder`. Later on we'll deprecate the `Ordinal` versions in favor of these. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-order
label:t-algebra$
54/1 Mathlib/Algebra/Order/SuccPred.lean 1 2 ['github-actions', 'plp127'] nobody
133-63669
4 months ago
unknown
unknown
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
133-37345
4 months ago
unknown
unknown
27995 kckennylau
author:kckennylau
feat(RingTheory/Valuation): alternate constructors for Valuation --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
132-9220
4 months ago
144-67074
144 days ago
17-71108
17 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? [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-data large-import 220/3 Mathlib/Data/Real/Embedding.lean 1 2 ['github-actions', 'mathlib4-merge-conflict-bot'] nobody
131-14353
4 months ago
131-14354
131 days ago
40-31514
40 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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-algebra
label:t-algebra$
34/0 Mathlib/Algebra/QuadraticDiscriminant.lean 1 8 ['chrisflav', 'github-actions', 'tb65536', 'upobir'] chrisflav
assignee:chrisflav
130-68524
4 months ago
154-60052
154 days ago
55-8757
55 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 merge-conflict t-computability awaiting-author 120/0 Mathlib/Computability/Halting.lean 1 13 ['YaelDillies', 'github-actions', 'iehality', 'mathlib4-merge-conflict-bot'] YaelDillies
assignee:YaelDillies
129-898
4 months ago
148-83779
148 days ago
7-81013
7 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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-algebra
label:t-algebra$
41/0 Mathlib/Algebra/Order/Monoid/Canonical/Basic.lean 1 5 ['YaelDillies', 'github-actions', 'mathlib4-dependent-issues-bot', 'vihdzp'] nobody
128-71411
4 months ago
168-4075
168 days ago
0-41339
11 hours
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-category-theory 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
128-67580
4 months ago
128-67581
128 days ago
0-1045
17 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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-category-theory 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
128-62619
4 months ago
184-6321
184 days ago
0-51
51 seconds
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! [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-algebra new-contributor
label:t-algebra$
10/0 Mathlib/LinearAlgebra/Projection.lean 1 7 ['PSchwahn', 'github-actions', 'joelriou', 'kckennylau'] joelriou
assignee:joelriou
128-35429
4 months ago
128-66532
128 days ago
73-38219
73 days
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-category-theory 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
127-76470
4 months ago
unknown
unknown
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 --- merge-conflict t-logic new-contributor 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
127-70331
4 months ago
127-70332
127 days ago
10-49648
10 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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-differential-geometry new-contributor 36/0 Mathlib/Geometry/Manifold/ContMDiff/Defs.lean 1 13 ['bwangpj', 'girving', 'github-actions', 'grunweg', 'kbuzzard', 'sgouezel'] sgouezel
assignee:sgouezel
127-50184
4 months ago
128-4219
128 days ago
22-76960
22 days
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR t-meta 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
127-3495
4 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-category-theory 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
126-39655
4 months ago
unknown
unknown
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. WIP CI 475/0 scripts/README.md,scripts/check_github_urls.py 2 2 ['github-actions', 'kim-em'] nobody
126-28808
4 months ago
unknown
unknown
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) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-data 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
126-23297
4 months ago
177-18482
177 days ago
0-16748
4 hours
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-measure-probability new-contributor 8/0 Mathlib/MeasureTheory/Integral/Bochner/Set.lean 1 6 ['RemyDegenne', 'github-actions', 'sgouezel', 'thefundamentaltheor3m'] nobody
125-66053
4 months ago
216-73891
216 days ago
0-7890
2 hours
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) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-data large-import 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
125-38316
4 months ago
unknown
unknown
22517 j-loreaux
author:j-loreaux
feat: `ℕ+` powers in semigroups --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP large-import 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
124-43638
4 months ago
unknown
unknown
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. ------- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-data 459/212 Mathlib/Data/Ordmap/Ordnode.lean 1 4 ['eric-wieser', 'github-actions', 'grunweg', 'mathlib4-merge-conflict-bot'] nobody
124-20964
4 months ago
124-20965
124 days ago
39-68381
39 days
29615 eric-wieser
author:eric-wieser
chore: add a computable shortcut for `AddCommMonoid ℂ` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis easy bench-after-CI 9/1 Mathlib/Analysis/Complex/Basic.lean 1 1 ['github-actions'] nobody
123-84497
4 months ago
unknown
unknown
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). [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict large-import awaiting-CI t-meta 144/26 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Basic.lean,Mathlib/Tactic/TacticAnalysis/Declarations.lean,Mathlib/Tactic/TacticAnalysis/FunProp.lean,MathlibTest/TacticAnalysis2.lean 6 12 ['Vierkantor', 'github-actions', 'grunweg', 'mathlib4-merge-conflict-bot'] nobody
123-69622
4 months ago
unknown
unknown
29633 sgouezel
author:sgouezel
Just for bench --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
123-5206
4 months ago
unknown
unknown
25069 erdOne
author:erdOne
feat(EllipticCurve): rational points of singular nodal cubics --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-algebraic-geometry 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
122-58839
4 months ago
unknown
unknown
25070 erdOne
author:erdOne
feat(EllipticCurve): rational points on singular cuspidal cubics --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-algebraic-geometry 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
122-58838
4 months ago
unknown
unknown
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 merge-conflict awaiting-author t-algebra
label:t-algebra$
162/5 Mathlib.lean,Mathlib/GroupTheory/GroupExtension/Abelian.lean,Mathlib/GroupTheory/GroupExtension/Basic.lean,Mathlib/GroupTheory/GroupExtension/Defs.lean,docs/references.bib 5 3 ['erdOne', 'github-actions', 'mathlib4-merge-conflict-bot', 'yu-yama'] erdOne
assignee:erdOne
122-732
4 months ago
146-50510
146 days ago
49-14090
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 merge-conflict t-topology 651/0 Mathlib.lean,Mathlib/Topology/Algebra/FilterBasis.lean,Mathlib/Topology/Algebra/FilterBasisNew.lean,Mathlib/Topology/Algebra/Nonarchimedean/Bases.lean,Mathlib/Topology/Algebra/Nonarchimedean/BasesNew.lean 5 3 ['ADedecker', 'github-actions', 'mathlib4-merge-conflict-bot'] PatrickMassot
assignee:PatrickMassot
121-82575
3 months ago
121-82576
121 days ago
87-78694
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-differential-geometry 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
121-73232
3 months ago
153-59362
153 days ago
28-7893
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-order t-meta 14/16 Mathlib/Order/Filter/Defs.lean 1 2 ['github-actions', 'mathlib4-merge-conflict-bot'] nobody
121-71191
3 months ago
unknown
unknown
29605 alreadydone
author:alreadydone
experiment(Algebra): unbundle npow/zpow from Monoid/InvDivMonoid --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra awaiting-CI
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
121-61826
3 months ago
unknown
unknown
29614 sgouezel
author:sgouezel
Sg test4 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
120-72753
3 months ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-data 33/36 Mathlib/Algebra/Order/Archimedean/Basic.lean,Mathlib/Algebra/Order/Sub/Defs.lean,Mathlib/Algebra/Polynomial/Derivative.lean,Mathlib/AlgebraicGeometry/EllipticCurve/DivisionPolynomial/Degree.lean,Mathlib/Analysis/Asymptotics/Lemmas.lean,Mathlib/Analysis/Complex/UpperHalfPlane/Metric.lean,Mathlib/Combinatorics/Hall/Finite.lean,Mathlib/Combinatorics/SimpleGraph/Copy.lean,Mathlib/Combinatorics/SimpleGraph/Regularity/Uniform.lean,Mathlib/Data/Finset/Card.lean,Mathlib/Data/Nat/Squarefree.lean,Mathlib/MeasureTheory/Integral/Bochner/VitaliCaratheodory.lean,Mathlib/RingTheory/Polynomial/Pochhammer.lean,Mathlib/Topology/ContinuousMap/Polynomial.lean 14 10 ['JovanGerb', 'eric-wieser', 'github-actions', 'mathlib4-merge-conflict-bot'] nobody
120-69470
3 months ago
unknown
unknown
29010 grunweg
author:grunweg
chore: more tests for field_simp features and edge cases --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 135/0 MathlibTest/FieldSimp.lean 1 2 ['github-actions', 'mathlib4-merge-conflict-bot'] nobody
120-49035
3 months ago
140-20886
140 days ago
0-69174
19 hours
27937 madvorak
author:madvorak
feat(Logic/Basic): `congr_heq₂` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-logic 6/0 Mathlib/Logic/Basic.lean 1 8 ['YaelDillies', 'fpvandoorn', 'github-actions', 'madvorak', 'vihdzp'] fpvandoorn
assignee:fpvandoorn
119-85768
3 months ago
146-153
145 days ago
17-59565
17 days
29741 JovanGerb
author:JovanGerb
trying #28803 using lean#10178 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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 2 ['JovanGerb', 'leanprover-bot'] nobody
119-81377
3 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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
119-67979
3 months ago
unknown
unknown
7125 eric-wieser
author:eric-wieser
feat: additive monoid structure via biproducts I suspect I'm missing a trick with these transport lemmas. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-category-theory awaiting-CI 237/0 Mathlib/CategoryTheory/Limits/Skeleton.lean 1 3 ['alreadydone', 'eric-wieser', 'mathlib4-merge-conflict-bot'] nobody
119-44296
3 months ago
unknown
unknown
27950 alreadydone
author:alreadydone
feat(MonoidAlgebra): criteria for `single` to be a unit, irreducible or prime --- - [ ] depends on: #27936 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-algebra blocked-by-other-PR
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 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
118-75360
3 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
116-77495
3 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-category-theory 118/0 Mathlib/CategoryTheory/Adhesive.lean 1 1 ['github-actions'] nobody
115-38787
3 months ago
unknown
unknown
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.) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-category-theory 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
114-53861
3 months ago
129-2194
129 days ago
13-47821
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-algebra large-import
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
113-9661
3 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-group-theory 61/68 Mathlib/GroupTheory/Perm/Fin.lean 1 10 ['JovanGerb', 'eric-wieser', 'github-actions', 'mathlib4-merge-conflict-bot', 'plp127', 'tb65536'] nobody
113-7772
3 months ago
113-7773
113 days ago
19-72402
19 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. awaiting-author t-analysis new-contributor 383/0 Mathlib/Analysis/Complex/Residue/Basic.lean 1 17 ['Periecle', 'github-actions', 'hrmacbeth', 'llllvvuu', 'loefflerd'] nobody
112-69531
3 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra
label:t-algebra$
177/122 Mathlib/Algebra/Group/Action/Defs.lean,Mathlib/Algebra/Group/Basic.lean,Mathlib/Algebra/Group/Commute/Defs.lean,Mathlib/Algebra/Group/Defs.lean,Mathlib/Algebra/Group/Ext.lean,Mathlib/Algebra/Group/Int/Defs.lean,Mathlib/Algebra/Group/Opposite.lean,Mathlib/Algebra/Group/Pointwise/Set/Basic.lean,Mathlib/Algebra/Group/Prod.lean,Mathlib/Algebra/Group/Submonoid/Membership.lean,Mathlib/Algebra/Group/TypeTags/Basic.lean,Mathlib/Algebra/Group/Units/Defs.lean,Mathlib/Algebra/GroupWithZero/Basic.lean,Mathlib/Algebra/Module/NatInt.lean,Mathlib/Algebra/Order/GroupWithZero/Unbundled/Basic.lean,Mathlib/Algebra/Order/Monoid/Unbundled/WithTop.lean,Mathlib/Algebra/Order/Ring/Unbundled/Basic.lean,Mathlib/Algebra/Ring/ULift.lean,Mathlib/Data/BitVec.lean,Mathlib/Tactic/Abel.lean,Mathlib/Tactic/NormNum/Pow.lean 21 2 ['github-actions', 'mathlib4-merge-conflict-bot'] nobody
112-18030
3 months ago
unknown
unknown
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebraic-geometry blocked-by-other-PR RFC 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
112-1860
3 months ago
unknown
unknown
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-category-theory new-contributor 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
111-70362
3 months ago
unknown
unknown
27829 dupuisf
author:dupuisf
feat: modify `cfc_tac` to use `grind` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
110-72273
3 months ago
unknown
unknown
21950 erdOne
author:erdOne
feat(NumberTheory/Padics): the completion of `ℚ` at a finite place is `ℚ_[p]` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-number-theory 253/1 Mathlib.lean,Mathlib/Algebra/GroupWithZero/WithZero.lean,Mathlib/NumberTheory/Padics/HeightOneSpectrum.lean,Mathlib/NumberTheory/Padics/PadicNumbers.lean,Mathlib/Topology/Algebra/Valued/WithVal.lean,Mathlib/Topology/Algebra/WithZeroMulInt.lean,Mathlib/Topology/Algebra/WithZeroTopology.lean 7 33 ['Ruben-VandeVelde', 'erdOne', 'faenuccio', 'github-actions', 'leanprover-community-bot-assistant', 'pechersky', 'smmercuri', 'xroblot'] nobody
110-69282
3 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-combinatorics 76/0 Mathlib/Combinatorics/SimpleGraph/Metric.lean 1 3 ['github-actions', 'leanprover-community-mathlib4-bot', 'mathlib4-merge-conflict-bot'] nobody
108-71244
3 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author new-contributor t-measure-probability 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
108-42430
3 months ago
139-255
139 days ago
0-22659
6 hours
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-category-theory new-contributor 17/0 Mathlib/CategoryTheory/Limits/Shapes/Products.lean 1 6 ['chrisflav', 'github-actions', 'leanprover-community-bot-assistant', 'ppls-nd-prs', 'robin-carlier'] nobody
107-84575
3 months ago
209-7575
209 days ago
0-45487
12 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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-category-theory 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
107-59364
3 months ago
107-59365
107 days ago
0-4044
1 hour
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR t-category-theory 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
107-59362
3 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR t-category-theory 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
107-59360
3 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR t-category-theory large-import 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
107-59358
3 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR t-category-theory large-import 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 4 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
107-59233
3 months ago
168-65096
168 days ago
0-898
14 minutes
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR t-category-theory large-import 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 4 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
107-59231
3 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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR t-category-theory large-import 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 4 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
107-59230
3 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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR t-category-theory large-import 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 4 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
107-59228
3 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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR t-category-theory large-import 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 4 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
107-59226
3 months ago
167-83987
167 days ago
0-3210
53 minutes
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR t-category-theory large-import 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
107-59225
3 months ago
unknown
unknown
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 awaiting-author t-data 360/0 MathlibTest/Junk.lean 1 17 ['SnirBroshi', 'Timeroot', 'bryangingechen', 'github-actions', 'leanprover-community-bot-assistant', 'madvorak', 'pechersky', 'vihdzp'] pechersky
assignee:pechersky
107-26609
3 months ago
107-26609
107 days ago
33-15711
33 days
28452 plp127
author:plp127
feat: Define `ZMod.fintype` without cases Define `ZMod.fintype` without casing on `n` except inside the proof. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-data 2/3 Mathlib/Data/ZMod/Defs.lean 1 2 ['github-actions', 'jcommelin'] pechersky
assignee:pechersky
107-25828
3 months ago
107-25828
107 days ago
45-84688
45 days
28807 alreadydone
author:alreadydone
experiment: Submodule with SMul only (no Semiring) --- `SubMulAction` already takes `SMul`. TODO: relax typeclass requirements of `Ideal` as well. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra awaiting-CI bench-after-CI
label:t-algebra$
54/42 Mathlib/Algebra/Module/Submodule/Defs.lean 1 2 ['github-actions', 'mathlib4-merge-conflict-bot'] nobody
107-22398
3 months ago
unknown
unknown
28808 alreadydone
author:alreadydone
experiment: Ideal with Mul only (no Semiring) --- - [ ] depends on: #28807 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra blocked-by-other-PR bench-after-CI awaiting-CI merge-conflict
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
107-22397
3 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebraic-topology t-category-theory 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
106-78766
3 months ago
201-86050
201 days ago
0-1046
17 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) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
106-45133
3 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR t-category-theory large-import 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
105-85630
3 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-category-theory large-import 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
105-81991
3 months ago
unknown
unknown
26115 grunweg
author:grunweg
WIP/proof of concept,feat: the inverse function theorem for manifolds --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-differential-geometry 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
104-83878
3 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR t-analysis 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
104-81387
3 months ago
155-67485
155 days ago
13-34998
13 days
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP blocked-by-other-PR t-category-theory awaiting-CI large-import merge-conflict 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
104-50502
3 months ago
unknown
unknown
30079 dagurtomas
author:dagurtomas
feat(CategoryTheory): IsSheafFor as a multiequalizer condition --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-category-theory 112/0 Mathlib/CategoryTheory/Sites/Multifork.lean 1 3 ['chrisflav', 'github-actions', 'joelriou'] nobody
104-37826
3 months ago
unknown
unknown
29012 grunweg
author:grunweg
chore: reduce `Topology` imports in `Data` Move Data.Real.Sqrt to Analysis. --- - [ ] depends on: #28966 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict file-removed 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
103-77304
3 months ago
unknown
unknown
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) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-category-theory 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
103-65105
3 months ago
unknown
unknown
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`. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-algebra
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
103-372
3 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) --- *This PR continues the work from #21747.* *Original PR: https://github.com/leanprover-community/mathlib4/pull/21747* merge-conflict t-algebraic-topology blocked-by-other-PR large-import 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
102-86006
3 months ago
unknown
unknown
23621 astrainfinita
author:astrainfinita
chore: deprecate `LinearOrderedComm{Monoid, Group}WithZero` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) - [x] depends on: #20676 merge-conflict t-algebra t-order
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 24 ['YaelDillies', 'astrainfinita', 'github-actions', 'grunweg', 'leanprover-bot', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] kbuzzard
assignee:kbuzzard
102-63706
3 months ago
unknown
unknown
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) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) IMO awaiting-author new-contributor 196/0 Archive.lean,Archive/Imo/Imo1975Q3.lean 2 36 ['Antidite', 'LLaurance', 'github-actions', 'jsm28'] jsm28
assignee:jsm28
102-50321
3 months ago
102-50321
102 days ago
46-21614
46 days
30192 erdOne
author:erdOne
feat(RingTheory): valuative topology = adic topology for discrete rank 1 valuations --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-ring-theory t-topology 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
101-79429
3 months ago
unknown
unknown
26886 pechersky
author:pechersky
feat(NumberTheory/Padics/ValuativeRel): ValuativeRel ℚ_[p] as well as instances for IsRankLeOne, IsNontrivial, IsDiscrete --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) - [ ] depends on: #26827 WIP t-number-theory blocked-by-other-PR t-algebra merge-conflict t-analysis
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
101-36906
3 months ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-number-theory 139/0 Archive.lean,Archive/Examples/Local/Laurent.lean,Archive/Examples/Local/NumberField.lean,Archive/Examples/Local/Padic.lean,Archive/Examples/Local/Witt.lean 5 6 ['faenuccio', 'github-actions', 'mathlib4-merge-conflict-bot', 'riccardobrasca'] riccardobrasca
assignee:riccardobrasca
101-36664
3 months ago
101-36664
101 days ago
78-82075
78 days
27314 pechersky
author:pechersky
feat(TopologyValued): `Valued` based on a range topology Switch from a topology based on `fun γ : Γ₀ˣ => (v.ltAddSubgroup γ : AddSubgroup R)` to ``` fun rs : {rs : R × R // v rs.1 ≠ 0 ∧ v rs.2 ≠ 0} ↦ (v.ltAddSubgroup (Units.mk0 (v rs.val.2 / v rs.val.1) (by simp [rs.prop])) : AddSubgroup R) ``` This is in preparation for using `IsValuativeTopology` instead. In fact, that basis is precisely what `ValuativeTopology` asserts. `Valued.mk'` is kept, we do not yet rely on `IsValuativeTopology` and `UniformSpace`. The new `Valued` behaves the same way as it did before for `MulArchimedean` valuation codomains, which are all of the current in-mathlib uses of `Valued`. This is, for rank-one valuations. For valuations which rank one, but do not pass to the whole codomain, there are helper lemmas to discuss open/closed/clopen sets. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) - [x] depends on: #27264 - [x] depends on: #27265 - [ ] depends on: #27163 - [x] depends on: #27339 merge-conflict t-topology 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
100-69957
3 months ago
unknown
unknown
30135 erdOne
author:erdOne
feat(RingTheory): `ValuativeRel` on subrings --- @pechersky do we want this? [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-ring-theory 19/0 Mathlib/RingTheory/Valuation/ValuativeRel/Basic.lean 1 5 ['erdOne', 'github-actions', 'pechersky'] nobody
100-64002
3 months ago
101-36694
101 days ago
3-19285
3 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 merge-conflict awaiting-author t-ring-theory 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
100-54975
3 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
98-85635
3 months ago
98-85636
98 days ago
25-73895
25 days
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-differential-geometry 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
98-67820
3 months ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-differential-geometry blocked-by-other-PR 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
98-67696
3 months ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) - [ ] depends on: #28325 t-number-theory blocked-by-other-PR t-algebra large-import merge-conflict t-topology
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
96-81378
3 months ago
155-11940
155 days ago
0-846
14 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] --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR new-contributor 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
96-64841
3 months ago
unknown
unknown
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 merge-conflict t-category-theory new-contributor 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
96-60776
3 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author new-contributor t-measure-probability 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
96-59626
3 months ago
unknown
unknown
30359 JLimperg
author:JLimperg
[Not a PR] Benchmark for Aesop RPINF precompilation --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict file-removed 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
96-51633
3 months ago
unknown
unknown
30351 JLimperg
author:JLimperg
[Not a PR] Benchmark Aesop's lazy forward state construction Testing the performance impact of an Aesop change. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict dependency-bump 3/3 lake-manifest.json,lakefile.lean 2 11 ['JLimperg', 'github-actions', 'leanprover-bot', 'mathlib4-merge-conflict-bot'] nobody
96-40534
3 months ago
unknown
unknown
30425 JLimperg
author:JLimperg
[Not a PR] Benchmark Aesop with precompiled RPINF at instance transparency --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
96-33738
3 months ago
unknown
unknown
30438 JLimperg
author:JLimperg
[Not a PR] Benchmark Aesop change that computes fewer RPINFs --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
95-64115
3 months ago
unknown
unknown
30440 JLimperg
author:JLimperg
[Not a PR] Benchmark Aesop with no `hypTypes` in `ForwardState` and `instances` RPINF transparency --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
95-59596
3 months ago
unknown
unknown
30452 JLimperg
author:JLimperg
[Not a PR] Benchmark Aesop with no `hypTypes` in `ForwardState`, RPINF at `instances` transparency and lazy forward state --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
95-40475
3 months ago
unknown
unknown
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`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-data 95/0 Mathlib/Data/Nat/Factors.lean 1 11 ['b-mehta', 'github-actions', 'grunweg', 'plp127'] b-mehta
assignee:b-mehta
94-76504
3 months ago
95-17317
95 days ago
111-942
111 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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-ring-theory 172/0 Counterexamples.lean,Counterexamples/DiscreteTopologyWithNontrivialValuation.lean 2 14 ['github-actions', 'grunweg', 'kckennylau', 'mathlib4-merge-conflict-bot', 'pechersky'] nobody
94-65837
3 months ago
94-65838
94 days ago
67-78029
67 days
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-category-theory 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
94-62575
3 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-differential-geometry 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
94-2384
3 months ago
unknown
unknown
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) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-topology 250/76 Mathlib/Analysis/Normed/Group/Basic.lean,Mathlib/Analysis/Normed/Group/Hom.lean,Mathlib/Analysis/Normed/Group/SeparationQuotient.lean,Mathlib/Analysis/Normed/Module/RCLike/Real.lean,Mathlib/Analysis/Normed/Operator/Basic.lean,Mathlib/Analysis/Normed/Operator/NormedSpace.lean,Mathlib/Analysis/NormedSpace/Multilinear/Basic.lean,Mathlib/Topology/EMetricSpace/Basic.lean,Mathlib/Topology/Homeomorph/Defs.lean,Mathlib/Topology/Inseparable.lean,Mathlib/Topology/Maps/Basic.lean,Mathlib/Topology/Order.lean,Mathlib/Topology/Sets/Opens.lean,Mathlib/Topology/Sheaves/PUnit.lean 14 5 ['github-actions', 'mathlib4-merge-conflict-bot'] nobody
93-63136
3 months ago
unknown
unknown
26561 b-mehta
author:b-mehta
feat(LiminfLimsup): liminf of an antitone function is its supremum --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) - [x] depends on: #26560 help-wanted t-topology 24/0 Mathlib/Topology/Order/LiminfLimsup.lean 1 4 ['b-mehta', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
93-18962
3 months ago
192-50914
192 days ago
0-6
6 seconds
21853 smmercuri
author:smmercuri
feat: the adele ring of a number field is locally compact --- - [ ] depends on: #21158 - [ ] depends on: #21847 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-number-theory large-import 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
91-72699
2 months ago
unknown
unknown
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!) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-number-theory t-algebra awaiting-CI merge-conflict
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
91-67413
2 months ago
unknown
unknown
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). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-data 19/0 Mathlib/Data/Fintype/Quotient.lean 1 12 ['github-actions', 'kckennylau', 'pechersky', 'tristan-f-r', 'vihdzp'] pechersky
assignee:pechersky
91-17369
2 months ago
91-17369
91 days ago
5-78194
5 days
28925 grunweg
author:grunweg
chore: remove `linear_combination'` tactic When `linear_combination` was refactored in #15899, the old code was kept as the `linear_combination'` tactic, for easier migration. The consensus of the zulip discussion ([#mathlib4 > Narrowing the scope of `linear_combination` @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Narrowing.20the.20scope.20of.20.60linear_combination.60/near/470237816)) was to wait, and "revisit this once people have experienced the various tactics in practice". One year later, the old tactic has almost no uses: it is unused in mathlib; [searching on github](https://github.com/search?q=linear_combination%27%20path%3A*.lean&type=code) yields 37 hits --- all of which are in various forks of mathlib. Thus, removing this tactic seems appropriate. --- Do not merge before the zulip discussion has concluded! [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict file-removed awaiting-zulip 0/564 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/LinearCombination'.lean,Mathlib/Tactic/Linter/UnusedTactic.lean,MathlibTest/linear_combination'.lean 5 4 ['euprunin', 'github-actions', 'grunweg', 'mathlib4-merge-conflict-bot'] nobody
91-12445
2 months ago
unknown
unknown
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 ``` WIP t-meta 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
90-63763
2 months ago
unknown
unknown
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` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data t-order delegated easy 17/7 Mathlib/Combinatorics/Enumerative/Composition.lean,Mathlib/Data/Finset/Sort.lean 2 4 ['eric-wieser', 'github-actions', 'mathlib-bors', 'ocfnash'] nobody
90-50994
2 months ago
111-83084
111 days ago
3-76820
3 days
19616 adamtopaz
author:adamtopaz
fix: fix the definition of the absolute Galois group of a field Previously it was defined as the Galois group of the algebraic closure, as opposed to the separable closure. Also, this adds some missing instances for this group. Still missing is compactness, but that seems like a bigger project. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra awaiting-author t-number-theory
label:t-algebra$
23/8 Mathlib/FieldTheory/AbsoluteGaloisGroup.lean,Mathlib/FieldTheory/KrullTopology.lean 2 4 ['acmepjz', 'alreadydone', 'github-actions'] nobody
89-6216
2 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-category-theory awaiting-CI 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
89-1
2 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebraic-topology blocked-by-other-PR new-contributor 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
88-53957
2 months ago
158-64493
158 days ago
0-2143
35 minutes
16428 astrainfinita
author:astrainfinita
test use `QuotLike` APIs --- - [ ] depends on: #16421 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-data 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
88-14580
2 months ago
unknown
unknown
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) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict tech debt blocked-by-other-PR t-data 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
88-14579
2 months ago
unknown
unknown
30642 thorimur
author:thorimur
bench: lean4#10832 merge-conflict large-import 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
87-60790
2 months ago
unknown
unknown
30643 thorimur
author:thorimur
bench: before lean4#10832 merge-conflict large-import 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
87-60789
2 months ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-group-theory new-contributor 6/0 Mathlib/GroupTheory/GroupAction/CardCommute.lean 1 17 ['github-actions', 'kckennylau', 'plp127', 'tb65536'] tb65536
assignee:tb65536
86-69876
2 months ago
86-69876
86 days ago
8-4679
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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 delegated t-category-theory 182/2 Mathlib/AlgebraicTopology/SimplexCategory/GeneratorsRelations/NormalForms.lean 1 6 ['github-actions', 'joelriou', 'mathlib-bors', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
85-70664
2 months ago
86-62380
86 days ago
0-21238
5 hours
30209 Ruben-VandeVelde
author:Ruben-VandeVelde
feat: some TwoSidedIdeal.span lemmas --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-ring-theory FLT 16/0 Mathlib/RingTheory/TwoSidedIdeal/Operations.lean 1 2 ['erdOne', 'github-actions'] erdOne
assignee:erdOne
85-41170
2 months ago
85-41170
85 days ago
17-8026
17 days
25225 xcloudyunx
author:xcloudyunx
feat(Combinatorics/SimpleGraph): Eulerian walk in connected graph contains all vertices --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-combinatorics new-contributor 16/0 Mathlib/Combinatorics/SimpleGraph/Trails.lean 1 6 ['IvanRenison', 'github-actions', 'vlad902'] kmill
assignee:kmill
85-33408
2 months ago
unknown
unknown
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 = ⊤`. awaiting-author t-category-theory 48/2 Mathlib/CategoryTheory/Adjunction/PartialAdjoint.lean 1 1 ['github-actions'] nobody
84-65644
2 months ago
unknown
unknown
27196 YaelDillies
author:YaelDillies
refactor(Polynomial/Bivariate): swap `X` and `Y` for improved notation This way, `X` keeps on being `X`. From Toric --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-algebra toric
label:t-algebra$
3/3 Mathlib/Algebra/Polynomial/Bivariate.lean 1 7 ['YaelDillies', 'alreadydone', 'github-actions', 'kckennylau'] nobody
84-59197
2 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra
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
84-23258
2 months ago
unknown
unknown
27683 dupuisf
author:dupuisf
feat: grind tags for set operations This PR adds `grind` tags for various set operations (union, intersection, complement, etc). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-data 29/9 Mathlib/Data/Set/Basic.lean,Mathlib/Data/Set/Operations.lean 2 5 ['dupuisf', 'euprunin', 'github-actions', 'mathlib4-merge-conflict-bot'] nobody
83-60947
2 months ago
unknown
unknown
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`). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
83-56840
2 months ago
unknown
unknown
25978 Bergschaf
author:Bergschaf
feat(Order/Sublocale): Open Sublocales --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) - [x] depends on: #25089 merge-conflict t-order 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
83-54693
2 months ago
156-12569
156 days ago
0-1326
22 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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-analysis 158/0 Mathlib.lean,Mathlib/Algebra/BigOperators/Ring/Finset.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Bounds.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/SeriesBounds.lean 4 28 ['Parcly-Taxel', 'Ruben-VandeVelde', 'adomani', 'girving', 'github-actions', 'llllvvuu', 'mathlib4-merge-conflict-bot', 'urkud'] nobody
83-52330
2 months ago
131-52119
131 days ago
0-72293
20 hours
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) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-linter awaiting-zulip 1/1 Mathlib/Tactic/Linter/Style.lean 1 1 ['github-actions'] nobody
81-46569
2 months ago
unknown
unknown
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). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict documentation awaiting-author 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
81-512
2 months ago
154-86096
154 days ago
0-40320
11 hours
28737 astrainfinita
author:astrainfinita
refactor: deprecate `MulEquivClass` This PR continues the work from #18806. Original PR: https://github.com/leanprover-community/mathlib4/pull/18806 merge-conflict awaiting-author t-algebra
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
79-2927
2 months ago
142-49500
142 days ago
2-23111
2 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! [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-number-theory new-contributor large-import 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
79-2879
2 months ago
94-63955
94 days ago
47-56535
47 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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
78-83931
2 months ago
96-40240
96 days ago
0-1188
19 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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor merge-conflict file-removed awaiting-author t-topology 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
78-81009
2 months ago
99-63638
99 days ago
0-553
9 minutes
30303 franv314
author:franv314
chore(Topology/Instances): add deprecated module Add deprecated module to moved Cantor set file. --- - [ ] depends on: #30299 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR new-contributor 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
78-81007
2 months ago
99-61839
99 days ago
0-8
8 seconds
30900 vihdzp
author:vihdzp
feat: run-length encoding --- - [ ] depends on: #30898 Moved from #17105. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR t-data large-import 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
78-76002
2 months ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-algebra new-contributor
label:t-algebra$
47/0 Mathlib/Algebra/Group/Subgroup/Pointwise.lean 1 10 ['FrederickPu', 'eric-wieser', 'github-actions', 'plp127', 'tb65536'] nobody
78-69838
2 months ago
87-59872
87 days ago
0-40723
11 hours
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology 51/0 Mathlib/Topology/TODO.lean 1 3 ['github-actions', 'plp127', 'urkud'] nobody
78-60175
2 months 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 merge-conflict WIP t-number-theory 22/0 Mathlib/NumberTheory/NumberField/InfinitePlace/Ramification.lean 1 2 ['github-actions', 'mathlib4-merge-conflict-bot'] nobody
77-66849
2 months ago
unknown
unknown
30975 mariainesdff
author:mariainesdff
feat(Data/Finsupp/Defs): add Finsupp.restrict Co-authored by: @AntoineChambert-Loir --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-data 49/0 Mathlib/Data/Finsupp/Defs.lean 1 4 ['ADedecker', 'github-actions'] nobody
77-64975
2 months ago
77-64975
77 days ago
1-79516
1 day
26357 javra
author:javra
feat(CategoryTheory): linear categories as `ModuleCat R`-enriched categories Continues #23826. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-category-theory large-import 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
76-25444
2 months ago
120-52097
120 days ago
15-12054
15 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 please-adopt WIP t-differential-geometry merge-conflict 75/6 Mathlib/Geometry/Manifold/Diffeomorph.lean,Mathlib/Geometry/Manifold/LocalDiffeomorph.lean 2 3 ['github-actions', 'grunweg', 'mathlib4-merge-conflict-bot'] nobody
75-83847
2 months ago
unknown
unknown
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra delegated
label:t-algebra$
141/26 Mathlib.lean,Mathlib/Data/Quot.lean,Mathlib/Data/Setoid/Basic.lean,Mathlib/GroupTheory/Congruence/Defs.lean,Mathlib/GroupTheory/Congruence/GroupWithZero.lean 5 32 ['ADedecker', 'eric-wieser', 'github-actions', 'mathlib-bors', 'mathlib4-merge-conflict-bot', 'ocfnash'] ocfnash
assignee:ocfnash
75-72583
2 months ago
155-1718
155 days ago
27-80433
27 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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
75-69084
2 months ago
unknown
unknown
30790 urkud
author:urkud
chore: partially migrate from `ContinuousMap.continuous` ... to `map_continuous` or `by fun_prop`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
75-68387
2 months 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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-ring-theory 65/20 Mathlib/RingTheory/GradedAlgebra/HomogeneousLocalization.lean 1 5 ['github-actions', 'mariainesdff'] mariainesdff
assignee:mariainesdff
75-35989
2 months ago
78-79797
78 days ago
17-71546
17 days
30631 ADedecker
author:ADedecker
refactor: evaluation of power series in semirings --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
74-68337
2 months ago
unknown
unknown
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`. --- --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-algebra new-contributor
label:t-algebra$
94/0 Mathlib/LinearAlgebra/Matrix/Transvection.lean,MathlibTest/matrix.lean 2 3 ['github-actions', 'riccardobrasca', 'zach1502'] nobody
72-80530
2 months ago
72-80530
72 days ago
41-49475
41 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) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-topology 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
72-76825
2 months ago
79-63898
79 days ago
117-47311
117 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`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-topology 368/1 Mathlib/Order/Lattice.lean,Mathlib/Topology/CWComplex/Classical/Subcomplex.lean 2 19 ['ADedecker', 'github-actions', 'scholzhannah'] nobody
72-69511
2 months ago
72-69511
72 days ago
6-67158
6 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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-ring-theory 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
72-68107
2 months ago
149-4603
149 days ago
47-3670
47 days
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict file-removed 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
72-63099
2 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
72-50508
2 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-category-theory 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
72-46605
2 months ago
unknown
unknown
22361 rudynicolop
author:rudynicolop
feat(Computability/NFA): nfa closure properties Add the closure properties union, intersection and reversal for NFA. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-computability merge-conflict awaiting-author awaiting-zulip 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
72-22135
2 months ago
unknown
unknown
30158 nicolaviolette
author:nicolaviolette
feat: combinatorics simplegraph basic --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-combinatorics new-contributor 9/4 Mathlib/Combinatorics/SimpleGraph/Basic.lean 1 3 ['b-mehta', 'github-actions'] b-mehta
assignee:b-mehta
72-13660
2 months ago
72-13660
72 days ago
31-68997
31 days
27708 vihdzp
author:vihdzp
feat: unions and intersections of ordinals are ordinals As well as a bonus result `IsTransitive.empty_mem`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-set-theory 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
71-79263
2 months ago
156-31302
156 days ago
12-1110
12 days
30431 kckennylau
author:kckennylau
feat(RingTheory): a homogeneous submodule is the span of its homogeneous elements --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
71-76169
2 months ago
72-69434
72 days ago
23-20971
23 days
27229 WilliamCoram
author:WilliamCoram
feat(GroupTheory/DoubleCoset): multiple lemmas From FLT --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) FLT t-group-theory 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
71-68559
2 months ago
84-85290
84 days ago
92-33213
92 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}`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-topology 44/0 Mathlib/MeasureTheory/Constructions/UnitInterval.lean,Mathlib/Topology/UnitInterval.lean 2 9 ['gaetanserre', 'github-actions', 'j-loreaux', 'mathlib4-merge-conflict-bot', 'ocfnash'] j-loreaux
assignee:j-loreaux
71-68014
2 months ago
71-68489
71 days ago
94-79080
94 days
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict file-removed awaiting-author t-ring-theory 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
71-53855
2 months ago
89-82660
89 days ago
25-70535
25 days
28132 dupuisf
author:dupuisf
feat: preliminary `grind` tags for `IsUnit` This PR adds preliminary `grind` tags for the `IsUnit` predicate. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra
label:t-algebra$
61/17 Mathlib/Algebra/Group/Action/Units.lean,Mathlib/Algebra/Group/Units/Defs.lean,Mathlib/Algebra/GroupWithZero/Units/Basic.lean,Mathlib/Algebra/Ring/Units.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Order.lean,Mathlib/Analysis/SpecialFunctions/ContinuousFunctionalCalculus/Rpow/Basic.lean 6 3 ['github-actions', 'mathlib4-merge-conflict-bot'] kim-em
assignee:kim-em
71-42435
2 months ago
71-42436
71 days ago
80-71574
80 days
25903 pfaffelh
author:pfaffelh
feat(MeasureTheory): finite unions of sets in a semi-ring (in terms of measure theory) form a ring : Finite unions of sets in a semi-ring (in terms of measure theory) form a ring The set containing finite unions of sets in a semi-ring are a ring. Part of `MeasureTheory.SetSemiring` is moved to the new file `MeasureTheory.SetRing`. --- - [ ] depends on: #25902 [contains changes in `SetSemiring` as well] --- *This PR continues the work from #23117.* *Original PR: https://github.com/leanprover-community/mathlib4/pull/23117* merge-conflict blocked-by-other-PR large-import t-measure-probability 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 5 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
71-30147
2 months ago
149-40693
149 days ago
0-10110
2 hours
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict large-import 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
71-10158
2 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-algebraic-geometry large-import 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
70-83479
2 months ago
91-41259
91 days ago
1-29930
1 day
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] [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-order large-import 35/0 Mathlib/Order/Preorder/Chain.lean 1 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
69-62239
2 months ago
unknown
unknown
26901 5hv5hvnk
author:5hv5hvnk
feat: a simproc version of `compute_degree` Wrap `compute_degree` in a simproc for use by simp. Closes #22219. --- awaiting-CI new-contributor merge-conflict awaiting-author t-meta 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
69-60328
2 months ago
unknown
unknown
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP help-wanted t-analysis 249/0 Mathlib.lean,Mathlib/Analysis/NormedSpace/HahnBanach/Splits.lean 2 2 ['github-actions', 'mathlib4-merge-conflict-bot'] nobody
69-47091
2 months ago
unknown
unknown
26391 grunweg
author:grunweg
feat: immersed submanifolds Still under construction --- - [ ] depends on: #26087 - [ ] depends on: #23040 Better version of #24549. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-differential-geometry blocked-by-other-PR 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
69-47088
2 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
69-45856
2 months ago
unknown
unknown
31340 kim-em
author:kim-em
feat: helper script to summarize CI errors --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) CI 235/0 scripts/README.md,scripts/failing_ci.py 2 1 ['github-actions'] nobody
69-32010
2 months 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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
68-79401
2 months ago
unknown
unknown
31348 PatrickMassot
author:PatrickMassot
chore: fix a docstring typo --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) documentation awaiting-author t-analysis easy 1/1 Mathlib/Analysis/Calculus/Darboux.lean 1 3 ['ADedecker', 'dopamine333', 'github-actions'] nobody
68-71365
2 months ago
68-71365
68 days ago
0-20900
5 hours
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP blocked-by-other-PR t-combinatorics 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
68-3822
2 months ago
unknown
unknown
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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 t-category-theory merge-conflict awaiting-author infinity-cosmos 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
66-61666
2 months ago
147-54392
147 days ago
17-13365
17 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 merge-conflict WIP t-topology t-algebra
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
65-49107
2 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
64-83642
2 months ago
unknown
unknown
26827 pechersky
author:pechersky
feat(Analysis/Normed/ValuativeRel): helper instance for NormedField --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) - [x] depends on: #26713 - [x] depends on: #26826 merge-conflict t-algebra t-number-theory t-analysis
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
63-71039
2 months ago
63-71039
63 days ago
126-50240
126 days
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-ring-theory new-contributor 17/0 Mathlib/RingTheory/MvPolynomial/Homogeneous.lean 1 6 ['LiamSchilling', 'chrisflav', 'github-actions'] chrisflav
assignee:chrisflav
63-27376
2 months ago
113-84317
113 days ago
2-17024
2 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. merge-conflict t-data 35/0 Mathlib/Data/List/Scan.lean 1 11 ['ShreckYe', 'github-actions', 'mathlib4-merge-conflict-bot', 'themathqueen', 'vlad902'] pechersky
assignee:pechersky
63-27270
2 months ago
66-25001
66 days ago
74-48754
74 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` [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory large-import new-contributor merge-conflict awaiting-zulip t-meta 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
63-23319
2 months ago
103-1985
103 days ago
0-29227
8 hours
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR large-import new-contributor 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
63-23317
2 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR large-import new-contributor 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
63-23316
2 months ago
unknown
unknown
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 merge-conflict t-differential-geometry 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
62-83571
2 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-differential-geometry blocked-by-other-PR 766/0 Mathlib.lean,Mathlib/Geometry/Diffeology/Basic.lean,Mathlib/Geometry/Diffeology/Continuous.lean,docs/references.bib 4 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
62-83447
2 months ago
180-25635
180 days ago
0-782
13 minutes
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!` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-meta 320/17 Mathlib/Tactic/GCongr/Core.lean,MathlibTest/GConvert.lean 2 2 ['github-actions', 'mathlib4-merge-conflict-bot'] nobody
62-52464
2 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra large-import
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
61-83345
2 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) delegated t-data 5/0 Mathlib/Data/Int/ModEq.lean 1 3 ['fpvandoorn', 'github-actions', 'mathlib-bors'] nobody
61-82585
2 months ago
215-68865
215 days ago
1-17595
1 day
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 merge-conflict t-number-theory large-import 1013/15 Mathlib.lean,Mathlib/Analysis/Complex/IntegerCompl.lean,Mathlib/Analysis/Complex/UpperHalfPlane/Basic.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/Topology/Algebra/InfiniteSum/NatInt.lean 11 9 ['CBirkbeck', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
61-70257
2 months ago
unknown
unknown
28733 CBirkbeck
author:CBirkbeck
E2 s transform --- - [ ] depends on : #29115 - [ ] depends on: #27606 - [ ] depends on" #26014 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict large-import 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 5 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
61-68577
2 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR large-import 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 4 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
61-68569
2 months 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. merge-conflict awaiting-author tech debt t-analysis 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 10 ['ADedecker', 'b-mehta', 'github-actions', 'j-loreaux', 'mathlib4-merge-conflict-bot', 'mcdoll', 'plp127'] nobody
61-68332
2 months ago
64-55704
64 days ago
2-74132
2 days
30978 dagurtomas
author:dagurtomas
Draft: adic spaces --- This is work in progress, mostly ported from the perfectoid project [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict large-import 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
61-64018
2 months ago
unknown
unknown
31582 ADedecker
author:ADedecker
chore: more flavours of derivatives within the empty set --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
61-62988
2 months 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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR new-contributor t-measure-probability 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
60-65110
1 month ago
unknown
unknown
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... [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-differential-geometry 57/9 Mathlib/Geometry/Manifold/VectorBundle/LocalFrame.lean 1 3 ['github-actions', 'grunweg', 'mathlib4-merge-conflict-bot'] nobody
60-52356
1 month ago
unknown
unknown
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-ring-theory 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
59-58614
1 month ago
60-65996
60 days ago
36-29414
36 days
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
59-48551
1 month ago
unknown
unknown
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-bench t-linter large-import merge-conflict awaiting-author t-meta 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 71 ['Command-Master', 'Vierkantor', 'github-actions', 'grunweg', 'kmill', 'leanprover-bot', 'mathlib4-merge-conflict-bot', 'thorimur', 'urkud'] nobody
59-38623
1 month ago
unknown
unknown
30770 robertmaxton42
author:robertmaxton42
(WIP) Limits and Colimits in Quiv WIP PR for the oleans --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
59-22784
1 month ago
unknown
unknown
31593 Ruben-VandeVelde
author:Ruben-VandeVelde
feat: some lemmas about MonoidAlgebra --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-algebra
label:t-algebra$
26/0 Mathlib/Algebra/MonoidAlgebra/Basic.lean 1 5 ['github-actions', 'mathlib4-merge-conflict-bot', 'robin-carlier', 'themathqueen'] nobody
59-16434
1 month ago
61-72094
61 days ago
0-83359
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... [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
59-8724
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-bench t-differential-geometry 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
58-61699
1 month ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) - [x] depends on: #26834 - [ ] depends on : #30135 t-algebra t-number-theory t-topology
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
58-55580
1 month ago
58-68600
58 days ago
131-48563
131 days
26087 grunweg
author:grunweg
feat: a `SliceModel` typeclass for models with corners for embedded submanifolds We define a new typeclass to denote a model with corners which "embeds" into another one: there are an embedding of the underlying topological spaces and a continuous linear inclusion between the normed spaces, which are compatible with the maps given by the models with corners. This condition is used for defining smooth (immersed and embedded) submanifolds: for `M` to be a submanifold of `N`, to boot their models with corners should be slice models. This will be defined in a future PR. To prove this definition is workable, we construct many basic instances of slice models - each model with corners is one over itself - slice models are transitive - each model with corners I embeds into two products `I.prod J` and `J.prod I` - Euclidean n-half-space embeds into Euclidean n-space - a Euclidean n-quadrant embeds into Euclidean half-space (hence into Euclidean n-space) - if n\leq m, Euclidean n-space embeds into Euclidean m-space [zulip discussion](https://leanprover.zulipchat.com/#narrow/channel/116395-maths/topic/Infinite-dimensional.20manifolds/near/413117885) ----------- - [x] depends on: #26083 - [x] depends on: #26082 - [x] depends on: #26086 - [x] depends on: #25705 This PR continues the work from #25505. merge-conflict t-differential-geometry 229/0 Mathlib.lean,Mathlib/Geometry/Manifold/SliceModel.lean 2 4 ['github-actions', 'grunweg', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
58-42438
1 month ago
204-53784
204 days ago
0-10615
2 hours
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-computability merge-conflict awaiting-author awaiting-zulip 307/5 Mathlib/Computability/NFA.lean 1 27 ['TpmKranz', 'YaelDillies', 'dupuisf', 'github-actions', 'leanprover-community-bot-assistant', 'meithecatte', 'rudynicolop'] nobody
58-40451
1 month ago
unknown
unknown
12032 mcdoll
author:mcdoll
feat: delta distribution as a limit --- - [ ] depends on: #11496 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-analysis 58/0 Mathlib/Analysis/Distribution/DiracDelta.lean 1 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
58-23425
1 month ago
unknown
unknown
26240 grunweg
author:grunweg
perf(CommandLinterLinter): use Substring more Probably, these changes make little difference, but let's find out. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-linter RFC 14/15 Mathlib/Tactic/Linter/CommandStart.lean 1 6 ['github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'mathlib4-merge-conflict-bot'] joneugster
assignee:joneugster
57-78316
1 month ago
57-78317
57 days ago
150-49908
150 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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-algebra RFC
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
57-74197
1 month ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author CI 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
57-57265
1 month ago
unknown
unknown
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` :) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import merge-conflict file-removed awaiting-author t-meta 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
57-57264
1 month ago
175-68384
175 days ago
0-4550
1 hour
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict CI 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
57-57263
1 month ago
72-20745
72 days ago
41-46786
41 days
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] [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-computability merge-conflict awaiting-author awaiting-zulip 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
57-56692
1 month ago
unknown
unknown
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-computability merge-conflict awaiting-author awaiting-zulip 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
57-55782
1 month ago
unknown
unknown
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] --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-meta 205/0 Mathlib.lean,Mathlib/Lean/Meta/AppBuilder.lean 2 1 ['mathlib4-merge-conflict-bot'] nobody
57-8152
1 month ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-meta 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
57-8151
1 month ago
unknown
unknown
5863 eric-wieser
author:eric-wieser
feat: add elaborators for concrete matrices --- - [x] depends on: #5866 - [ ] depends on: #5897 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict help-wanted blocked-by-other-PR t-meta 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
57-8150
1 month ago
unknown
unknown
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP new-contributor merge-conflict help-wanted t-analysis 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
57-8149
1 month ago
unknown
unknown
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) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-algebra RFC
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
57-8146
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-meta 141/0 Mathlib.lean,Mathlib/Tactic/Common.lean,Mathlib/Tactic/Setm.lean,test/Setm.lean 4 4 ['mathlib4-merge-conflict-bot', 'thorimur'] nobody
57-8145
1 month ago
unknown
unknown
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) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-analysis 404/0 Mathlib.lean,Mathlib/Analysis/Calculus/Gradient/Lemmas.lean 2 31 ['chenyili0818', 'github-actions', 'jcommelin', 'mathlib4-merge-conflict-bot', 'sgouezel', 'winstonyin'] nobody
57-8021
1 month ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-category-theory 74/0 Mathlib.lean,Mathlib/Data/Fiber.lean 2 18 ['adri326', 'joelriou', 'mathlib4-merge-conflict-bot', 'sinhp'] nobody
57-8020
1 month ago
unknown
unknown
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`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP awaiting-author t-algebra
label:t-algebra$
573/0 Mathlib.lean,Mathlib/LinearAlgebra/CliffordAlgebra/Basis.lean 2 16 ['github-actions', 'mathlib4-merge-conflict-bot'] nobody
57-8016
1 month ago
unknown
unknown
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? --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-differential-geometry merge-conflict awaiting-author t-topology t-analysis 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
57-8015
1 month ago
unknown
unknown
10998 hmonroe
author:hmonroe
feat(Logic): Arithmetization of partial recursive functions (toward Gödel's first incompleteness theorem) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-logic 364/0 Mathlib.lean,Mathlib/Logic/Godel/PartArith.lean 2 4 ['Ruben-VandeVelde', 'YaelDillies', 'mathlib4-merge-conflict-bot'] nobody
57-8014
1 month ago
unknown
unknown
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) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-linter 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
57-7890
1 month ago
unknown
unknown
11991 adomani
author:adomani
draft: syntax data linter A linter that prints `SyntaxNodeKind`s and `Range`s for all the nodes of a command. See this [Zulip discussion](https://leanprover.zulipchat.com/#narrow/stream/217875-Is-there-code-for-X.3F/topic/undocumented.20things). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
57-7889
1 month ago
unknown
unknown
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). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-meta 161/0 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Suffa.lean,test/Suffa.lean 4 4 ['MoritzBeroRoos', 'YaelDillies', 'mathlib4-merge-conflict-bot'] nobody
57-7887
1 month ago
unknown
unknown
13442 dignissimus
author:dignissimus
feat: mabel tactic for multiplicative abelian groups Mabel tactic for multiplicative abelian groups (#10361) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor merge-conflict modifies-tactic-syntax awaiting-author help-wanted t-meta 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
57-7885
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-algebra new-contributor
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
57-7883
1 month ago
unknown
unknown
14345 digama0
author:digama0
feat: the Dialectica category is monoidal closed - [x] depends on: #14274 The monoidal closed structure of the Dialectica category. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-category-theory 252/0 Mathlib.lean,Mathlib/CategoryTheory/Dialectica/Closed.lean 2 4 ['github-actions', 'kim-em', 'leanprover-community-mathlib4-bot', 'mathlib4-merge-conflict-bot'] nobody
57-7760
1 month ago
unknown
unknown
14727 jjaassoonn
author:jjaassoonn
feat(RingTheory/Flat/CategoryTheory): a flat module has vanishing higher Tor groups [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-ring-theory 37/1 Mathlib/RingTheory/Flat/CategoryTheory.lean 1 4 ['github-actions', 'kim-em', 'mathlib4-merge-conflict-bot'] nobody
57-7758
1 month ago
unknown
unknown
14733 jjaassoonn
author:jjaassoonn
feat(RingTheory/Flat/CategoryTheory): a module is flat iff tensoring preserves finite limits --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-ring-theory 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
57-7756
1 month ago
unknown
unknown
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`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-category-theory 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
57-7755
1 month ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-category-theory new-contributor 112/0 Mathlib.lean,Mathlib/CategoryTheory/Sites/CoveringFamilies.lean 2 21 ['AnthonyBordg', 'adamtopaz', 'dagurtomas', 'github-actions', 'joelriou', 'mathlib4-merge-conflict-bot'] nobody
57-7754
1 month ago
unknown
unknown
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) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
57-7752
1 month ago
unknown
unknown
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author CI 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
57-7750
1 month ago
unknown
unknown
17587 kmill
author:kmill
feat: Sym2-as-Finset theory --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-data new-contributor 105/3 Mathlib/Combinatorics/SimpleGraph/Basic.lean,Mathlib/Combinatorics/SimpleGraph/Finite.lean,Mathlib/Data/Sym/Sym2.lean,Mathlib/RingTheory/Polynomial/Vieta.lean 4 11 ['FordUniver', 'YaelDillies', 'github-actions', 'kmill', 'mathlib4-merge-conflict-bot'] nobody
57-7600
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-algebra t-category-theory awaiting-CI merge-conflict awaiting-author
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
57-7599
1 month ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-computability new-contributor 526/0 Mathlib.lean,Mathlib/Computability/Timed/InsertionSort.lean,Mathlib/Computability/Timed/Merge.lean,Mathlib/Computability/Timed/MergeSort.lean,Mathlib/Computability/Timed/Split.lean 5 9 ['github-actions', 'mathlib4-merge-conflict-bot'] nobody
57-7598
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-logic 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
57-7596
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR t-logic 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
57-7594
1 month ago
unknown
unknown
19323 madvorak
author:madvorak
feat: Function to Sum decomposition --- Discussion: https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Function.20to.20Sum.20decomposition merge-conflict WIP t-data 50/0 Mathlib.lean,Mathlib/Data/Sum/Decompose.lean 2 3 ['github-actions', 'madvorak', 'mathlib4-merge-conflict-bot'] nobody
57-7593
1 month ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-meta 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
57-7592
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-order t-data merge-conflict t-algebraic-geometry 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
57-7591
1 month ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-meta large-import 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
57-7464
1 month ago
unknown
unknown
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] [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-algebra 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
57-7463
1 month ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-data 37/0 Mathlib/Data/Matrix/Invertible.lean 1 5 ['eric-wieser', 'github-actions', 'mathlib4-merge-conflict-bot'] nobody
57-7461
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-computability awaiting-zulip new-contributor 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
57-7460
1 month ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP large-import merge-conflict t-combinatorics t-logic 175/0 Mathlib/ModelTheory/Graph.lean,Mathlib/ModelTheory/Substructures.lean 2 2 ['github-actions', 'mathlib4-merge-conflict-bot'] nobody
57-7458
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-algebra t-category-theory
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
57-7457
1 month ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-computability 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
57-7456
1 month ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-computability blocked-by-other-PR 676/0 Mathlib.lean,Mathlib/Computability/QueryComplexity/Basic.lean,Mathlib/Computability/QueryComplexity/Defs.lean,Mathlib/Computability/QueryComplexity/Sort.lean 4 4 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
57-7454
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author large-import t-logic 102/0 Mathlib/ModelTheory/Bundled.lean 1 27 ['GabinKolly', 'Vierkantor', 'YaelDillies', 'github-actions', 'mathlib4-merge-conflict-bot'] nobody
57-7452
1 month ago
unknown
unknown
21277 GabinKolly
author:GabinKolly
feat(ModelTheory/PartialEquiv): Define the mapping of a self-partialEquiv through an embedding Define the mapping of a self-partialEquiv through an embedding and the notion of fully extendable partialEquiv. --- This is some preparatory work for #18876 - [ ] depends on: #21276 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR t-logic 215/5 Mathlib/ModelTheory/PartialEquiv.lean,Mathlib/ModelTheory/Substructures.lean 2 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
57-7450
1 month ago
unknown
unknown
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-topology 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
57-7447
1 month ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-category-theory 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
57-7446
1 month ago
unknown
unknown
21829 Whysoserioushah
author:Whysoserioushah
feat(LinearAlgebra/TensorProduct/HomTensor): Add TensorProduct of Hom-modules Co-authored-by: Andrew Yang --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-algebra
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
57-7444
1 month ago
unknown
unknown
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`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra new-contributor awaiting-CI large-import merge-conflict
label:t-algebra$
169/0 Mathlib/Algebra/Free.lean 1 12 ['YaelDillies', 'github-actions', 'mathlib4-merge-conflict-bot'] nobody
57-7320
1 month ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-computability awaiting-author new-contributor 70/0 Mathlib.lean,Mathlib/Computability/PDA.lean 2 35 ['YaelDillies', 'github-actions', 'madvorak', 'mathlib4-merge-conflict-bot', 'shetzl'] nobody
57-7314
1 month ago
unknown
unknown
22194 eric-wieser
author:eric-wieser
feat: oracle computations (alternative) This explores a simpler version of #20924 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-computability 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
57-7311
1 month ago
unknown
unknown
22231 pechersky
author:pechersky
feat(Algebra/Valued): `AdicExpansion` initial defns --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra awaiting-author t-topology
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
57-7310
1 month ago
unknown
unknown
22232 pechersky
author:pechersky
feat(Algebra/Valued): `AdicExpansion.apprUpto` --- - [ ] depends on: #22231 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-topology 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
57-7308
1 month ago
unknown
unknown
22233 pechersky
author:pechersky
feat(Algebra/Valued): `AdicExpansion.evalAt` --- - [ ] depends on: #22231 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-topology 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
57-7307
1 month ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-category-theory new-contributor 312/0 Mathlib.lean,Mathlib/CategoryTheory/Topos/Power.lean 2 3 ['github-actions', 'joelriou', 'mathlib4-merge-conflict-bot'] b-mehta
assignee:b-mehta
57-7305
1 month ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-computability awaiting-author new-contributor 383/0 Mathlib.lean,Mathlib/Computability/LeftmostDerivation.lean 2 55 ['YaelDillies', 'github-actions', 'madvorak', 'mathlib4-merge-conflict-bot', 'shetzl'] YaelDillies
assignee:YaelDillies
57-7303
1 month ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-linter large-import 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
57-7301
1 month ago
unknown
unknown
22497 adomani
author:adomani
test: decl diff in lean Testing branch for #22464. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP CI test-ci 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
57-7299
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra
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
57-7298
1 month ago
unknown
unknown
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. merge-conflict awaiting-author t-analysis new-contributor 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
57-7292
1 month ago
unknown
unknown
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). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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. merge-conflict awaiting-author t-algebra
label:t-algebra$
100/0 Mathlib.lean,Mathlib/LinearAlgebra/BilinearForm/Trace.lean 2 4 ['github-actions', 'jcommelin', 'mathlib4-merge-conflict-bot'] nobody
57-7290
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-data 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
57-7288
1 month ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-ring-theory 214/16 Mathlib/Algebra/RingQuot.lean,Mathlib/GroupTheory/Congruence/Hom.lean,Mathlib/RingTheory/Congruence/Defs.lean,Mathlib/RingTheory/Congruence/Hom.lean,Mathlib/RingTheory/TwoSidedIdeal/Kernel.lean 5 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-merge-conflict-bot'] nobody
57-7287
1 month ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-algebra t-category-theory large-import merge-conflict
label:t-algebra$
111/45 Mathlib/Order/DirectedInverseSystem.lean 1 2 ['github-actions', 'mathlib4-merge-conflict-bot'] nobody
57-7281
1 month ago
unknown
unknown
23460 Timeroot
author:Timeroot
feat: Definition of `Clone` Basics about Clones. Part of #20051 --- - [ ] depends on: #26329 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra blocked-by-other-PR
label:t-algebra$
326/0 Mathlib.lean,Mathlib/Algebra/Clone/Basic.lean,Mathlib/Algebra/Clone/Defs.lean,Mathlib/Data/Fin/Basic.lean 4 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
57-7279
1 month ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-topology large-import 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
57-7277
1 month ago
unknown
unknown
23585 plp127
author:plp127
feat: `Filter.atMax` and `Filter.atMin` Adds `atMax` and `atMin`, filters. Making an analogy, `atMax` : `atTop` :: `IsMax` : `IsTop`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-order 148/0 Mathlib.lean,Mathlib/Order/Filter/AtMaxMin.lean 2 5 ['github-actions', 'mathlib4-merge-conflict-bot', 'plp127', 'urkud'] nobody
57-7276
1 month ago
unknown
unknown
23758 erdOne
author:erdOne
feat(Topology/Algebra): linearly topologized iff non-archimedean ...for topological modules over compact rings or `ℤ`-finite rings --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra large-import merge-conflict awaiting-author t-topology
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
57-7274
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-topology 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
57-7272
1 month ago
85-847
85 days ago
64-67198
64 days
24161 urkud
author:urkud
feat(Analysis/Calculus/Schwarzian): new file --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-analysis 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
57-7140
1 month ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-combinatorics new-contributor 187/0 Mathlib.lean,Mathlib/Combinatorics/SimpleGraph/Cycle.lean 2 42 ['IvanRenison', 'github-actions', 'mathlib4-merge-conflict-bot', 'vlad902'] kmill
assignee:kmill
57-7139
1 month ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-category-theory 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
57-7134
1 month ago
unknown
unknown
24744 Timeroot
author:Timeroot
Post's lattice Draft PR for now so I can get CI checks. Eventually want to prove Post's Lattice --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
57-7129
1 month ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) - [x] depends on: #23111 merge-conflict t-topology 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
57-7126
1 month ago
57-7127
57 days ago
162-10999
162 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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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) merge-conflict awaiting-author t-algebra t-data
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
57-7121
1 month ago
107-27392
107 days ago
19-24554
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-analysis 141/0 Mathlib.lean,Mathlib/Analysis/PDE/Quasilinear/Defs.lean 2 2 ['github-actions', 'mathlib4-merge-conflict-bot'] nobody
57-7120
1 month ago
unknown
unknown
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) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-linter 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
57-6994
1 month ago
unknown
unknown
25683 eric-wieser
author:eric-wieser
feat: Enumeration of NonemptyInterval --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-data large-import 52/4 Mathlib/Data/Sym/Sym2/Fin.lean,Mathlib/Data/Sym/Sym2/Order.lean 2 2 ['github-actions', 'mathlib4-merge-conflict-bot'] nobody
57-6991
1 month ago
unknown
unknown
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. merge-conflict awaiting-author t-number-theory new-contributor 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
57-6990
1 month ago
unknown
unknown
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) --- *This PR continues the work from #24452.* *Original PR: https://github.com/leanprover-community/mathlib4/pull/24452* merge-conflict awaiting-author t-category-theory t-meta 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
57-6988
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) --- *This PR continues the work from #24454.* *Original PR: https://github.com/leanprover-community/mathlib4/pull/24454* WIP blocked-by-other-PR t-category-theory merge-conflict awaiting-author t-meta 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
57-6987
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) --- *This PR continues the work from #24506.* *Original PR: https://github.com/leanprover-community/mathlib4/pull/24506* merge-conflict blocked-by-other-PR t-meta 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
57-6985
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) --- *This PR continues the work from #24633.* *Original PR: https://github.com/leanprover-community/mathlib4/pull/24633* merge-conflict blocked-by-other-PR t-category-theory t-meta 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
57-6983
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) --- *This PR continues the work from #24634.* *Original PR: https://github.com/leanprover-community/mathlib4/pull/24634* merge-conflict blocked-by-other-PR t-category-theory t-meta 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
57-6982
1 month ago
unknown
unknown
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) --- *This PR continues the work from #24650.* *Original PR: https://github.com/leanprover-community/mathlib4/pull/24650* merge-conflict blocked-by-other-PR t-meta 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
57-6980
1 month ago
unknown
unknown
25838 Bergschaf
author:Bergschaf
feat(Order/Atoms): Finsets are Atomistic --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-order large-import 31/0 Mathlib/Order/Atoms.lean 1 2 ['github-actions', 'mathlib4-merge-conflict-bot'] nobody
57-6969
1 month ago
unknown
unknown
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 merge-conflict t-topology large-import 174/5 Mathlib/Topology/Compactness/CompactlyCoherentSpace.lean 1 5 ['github-actions', 'joelriou', 'mathlib4-merge-conflict-bot', 'scholzhannah'] ADedecker
assignee:ADedecker
57-6958
1 month ago
57-6959
57 days ago
147-61529
147 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 merge-conflict t-algebraic-geometry 0/12 Mathlib.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Group.lean 2 4 ['Multramate', 'github-actions', 'grunweg', 'mathlib4-merge-conflict-bot'] nobody
57-6957
1 month 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 merge-conflict awaiting-author t-number-theory 259/37 Mathlib/NumberTheory/EllipticDivisibilitySequence.lean 1 9 ['MichaelStollBayreuth', 'Multramate', 'github-actions', 'mathlib4-merge-conflict-bot', 'tb65536'] tb65536
assignee:tb65536
57-6955
1 month ago
unknown
unknown
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 merge-conflict t-number-theory 265/45 Mathlib/NumberTheory/EllipticDivisibilitySequence.lean 1 3 ['Multramate', 'github-actions', 'mathlib4-merge-conflict-bot'] nobody
57-6954
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-group-theory large-import 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
57-6949
1 month ago
184-753
184 days ago
9-85141
9 days
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-algebraic-geometry blocked-by-other-PR 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
57-6947
1 month ago
100-38044
100 days ago
110-40398
110 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 merge-conflict awaiting-author t-number-theory 101/4 Mathlib/NumberTheory/Divisors.lean 1 37 ['MichaelStollBayreuth', 'github-actions', 'mathlib4-merge-conflict-bot', 'upobir'] mariainesdff
assignee:mariainesdff
57-6804
1 month ago
163-69942
163 days ago
45-75114
45 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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR new-contributor t-measure-probability 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
57-6802
1 month ago
194-1808
194 days ago
15-66961
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR new-contributor t-measure-probability 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
57-6801
1 month ago
194-1756
194 days ago
15-65730
15 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`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) --- *This PR continues the work from #24838.* *Original PR: https://github.com/leanprover-community/mathlib4/pull/24838* merge-conflict awaiting-author t-measure-probability 198/2 Mathlib/MeasureTheory/Measure/TightNormed.lean 1 2 ['github-actions', 'mathlib4-merge-conflict-bot'] nobody
57-6782
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) --- *This PR continues the work from #24949.* *Original PR: https://github.com/leanprover-community/mathlib4/pull/24949* merge-conflict WIP t-measure-probability 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
57-6780
1 month ago
unknown
unknown
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`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP awaiting-author t-linter 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
57-6779
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP new-contributor merge-conflict awaiting-author t-analysis 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
57-6778
1 month ago
153-55168
153 days ago
44-74030
44 days
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-algebra awaiting-CI
label:t-algebra$
100/0 Mathlib.lean,Mathlib/Algebra/Clone/Defs.lean 2 4 ['Timeroot', 'YaelDillies', 'github-actions', 'mathlib4-merge-conflict-bot'] nobody
57-6774
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) please-adopt merge-conflict t-logic 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
57-6761
1 month ago
78-82626
78 days ago
87-74589
87 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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR t-logic 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
57-6760
1 month ago
unknown
unknown
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 merge-conflict t-data 201/0 Mathlib.lean,Mathlib/Data/Nat/LogFueled.lean 2 3 ['AntoineChambert-Loir', 'github-actions', 'mathlib4-merge-conflict-bot'] nobody
57-6759
1 month ago
unknown
unknown
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. merge-conflict awaiting-author t-algebra new-contributor
label:t-algebra$
465/0 Mathlib.lean,Mathlib/Algebra/Polynomial/ZMod.lean 2 3 ['Ruben-VandeVelde', 'github-actions', 'mathlib4-merge-conflict-bot'] nobody
57-6630
1 month ago
172-50388
172 days ago
25-4678
25 days
26644 kckennylau
author:kckennylau
feat(SetTheory/ZFC): Define the language of sets and state the ZFC axioms --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-set-theory 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
57-6628
1 month ago
143-57891
143 days ago
40-44014
40 days
26648 eric-wieser
author:eric-wieser
chore(TensorProduct): remove more `suppress_compilation`s --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-core-PR t-algebra
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
57-6627
1 month ago
193-8662
193 days ago
3-19470
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-category-theory new-contributor 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
57-6625
1 month ago
86-59644
86 days ago
61-75483
61 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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-analysis 341/0 Mathlib.lean,Mathlib/Analysis/Calculus/PartialDerivativeTest.lean 2 13 ['bjoernkjoshanssen', 'github-actions', 'j-loreaux', 'mathlib4-merge-conflict-bot', 'themathqueen'] nobody
57-6621
1 month ago
188-22410
188 days ago
4-42147
4 days
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-algebra 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
57-6605
1 month ago
unknown
unknown
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`) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-data 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
57-6604
1 month ago
57-6605
57 days ago
133-15886
133 days
26920 yuma-mizuno
author:yuma-mizuno
feat(Tactic.CategoryTheory): add associator inserting tactic --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-category-theory t-meta 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
57-6603
1 month ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) - [x] depends on: #26939 - [x] depends on: #26940 - [x] depends on: #26941 merge-conflict t-ring-theory blocked-by-other-PR t-order 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
57-6600
1 month ago
153-65286
153 days ago
10-59532
10 days
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 merge-conflict WIP t-category-theory 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
57-6593
1 month ago
unknown
unknown
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! --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-algebra
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
57-6590
1 month ago
168-49260
168 days ago
16-81051
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-combinatorics new-contributor 1266/0 Mathlib.lean,Mathlib/Combinatorics/SimpleGraph/Triangle/IndependenceNumber.lean 2 10 ['Pjotr5', 'github-actions', 'grunweg', 'mathlib4-merge-conflict-bot'] nobody
57-6588
1 month ago
unknown
unknown
27163 pechersky
author:pechersky
feat(Topology/ValuativeRel): of and to basis of compatible valuations --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) - [x] depends on: #30262 t-number-theory t-algebra merge-conflict awaiting-author t-topology
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
57-6587
1 month ago
58-38378
58 days ago
62-47306
62 days
27187 Komyyy
author:Komyyy
feat: `NONote` represents ordinals < ε₀ --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-set-theory 186/12 Mathlib/SetTheory/Ordinal/Notation.lean 1 3 ['github-actions', 'mathlib4-merge-conflict-bot', 'vihdzp'] nobody
57-6586
1 month ago
unknown
unknown
27215 kckennylau
author:kckennylau
feat(AlgebraicGeometry): Define the Zariski site on `CommRingCatᵒᵖ` We define the Zariski site on `CommRingCatᵒᵖ` by inducing the topology from `Scheme`, and then we show that this topology is equal to the one generated by the pretopology of finite, surjective, and standard open morphisms. --- - [x] depends on: #28614 - [x] depends on: #28615 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-algebraic-geometry 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
57-6585
1 month ago
113-85549
113 days ago
3-67449
3 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 merge-conflict awaiting-author t-ring-theory 391/0 Mathlib.lean,Mathlib/Algebra/Algebra/Equiv.lean,Mathlib/Algebra/DirectSum/Basic.lean,Mathlib/Algebra/DirectSum/Module.lean,Mathlib/Algebra/Module/LinearMap/Defs.lean,Mathlib/Algebra/Ring/Equiv.lean,Mathlib/Algebra/RingQuot.lean,Mathlib/RingTheory/GradedAlgebra/Basic.lean,Mathlib/RingTheory/GradedAlgebra/HomogeneousRelation.lean 9 17 ['chrisflav', 'erdOne', 'eric-wieser', 'github-actions', 'mathlib4-merge-conflict-bot', 'ocfnash', 'xyzw12345'] mattrobball
assignee:mattrobball
57-6455
1 month ago
60-59073
60 days ago
72-57461
72 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) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-category-theory 218/0 Mathlib.lean,Mathlib/CategoryTheory/Comma/Presheaf/LeftExtension.lean 2 4 ['erdOne', 'github-actions', 'mathlib4-merge-conflict-bot', 'robin-carlier'] erdOne
assignee:erdOne
57-6454
1 month ago
162-83053
162 days ago
15-67997
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) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-category-theory awaiting-CI 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
57-6452
1 month ago
141-8876
141 days ago
18-80250
18 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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-order 394/0 Mathlib.lean,Mathlib/Order/SigmaCompleteLattice.lean 2 9 ['PierreQuinton', 'YaelDillies', 'github-actions', 'mathlib4-merge-conflict-bot', 'vihdzp'] YaelDillies
assignee:YaelDillies
57-6449
1 month ago
162-61309
162 days ago
12-23596
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 merge-conflict WIP t-analysis large-import 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
57-6445
1 month ago
141-47336
141 days ago
30-61786
30 days
27534 PierreQuinton
author:PierreQuinton
feat: a typeclass for `sSup`/`sInf` to be lawful Adds lawful infima and suprema type classes. A preorder with lawful suprema: whenever a set has a least upper bound, `sSup` returns a least upper bound for that set. A preorder with lawful infima: whenever a set has a greatest lower bound, `sInf` returns a greastest lower bound for that set. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-order 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
57-6441
1 month ago
57-6442
57 days ago
114-33795
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-category-theory new-contributor 70/1 Mathlib/CategoryTheory/Category/Factorisation.lean 1 13 ['YunkaiZhang233', 'b-mehta', 'github-actions', 'mathlib4-merge-conflict-bot', 'robin-carlier'] nobody
57-6433
1 month ago
167-63996
167 days ago
0-2875
47 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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-analysis 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
57-6432
1 month ago
71-53761
71 days ago
81-43915
81 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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-differential-geometry new-contributor 80/0 Mathlib.lean,Mathlib/Geometry/Manifold/ZeroDim.lean 2 14 ['fyqing', 'github-actions', 'grunweg', 'mathlib4-merge-conflict-bot', 'tb65536'] grunweg
assignee:grunweg
57-6431
1 month ago
166-38658
166 days ago
0-3675
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 merge-conflict awaiting-author t-algebra large-import
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
57-6305
1 month ago
111-17663
111 days ago
37-61659
37 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) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-differential-geometry 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
57-6304
1 month ago
unknown
unknown
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) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-ring-theory 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
57-6303
1 month ago
60-64317
60 days ago
99-20559
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`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-meta 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
57-6300
1 month ago
126-84169
126 days ago
23-18263
23 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. merge-conflict t-combinatorics new-contributor 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
57-6299
1 month ago
57-6300
57 days ago
99-48372
99 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 | |---|---| | image | image| In the after version, the extension names are all clickable. Similar to #21450. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-meta 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
57-6293
1 month ago
139-49580
139 days ago
15-70623
15 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` ] --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-topology t-order large-import 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
57-6292
1 month ago
61-60970
61 days ago
93-38369
93 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))`. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-meta 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
57-6289
1 month ago
63-84029
63 days ago
57-65706
57 days
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 merge-conflict blocked-by-other-PR t-combinatorics new-contributor 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
57-6285
1 month ago
unknown
unknown
28868 yury-harmonic
author:yury-harmonic
feat(Positive): add `OfNat` instance Also fix defeq for `Div` in the `Group` instance. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra large-import
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
57-6147
1 month ago
unknown
unknown
28871 JaafarTanoukhi
author:JaafarTanoukhi
feat(Combinatorics/Digraph): Tournaments Define orientations and tournaments. Related to #26771. Co-authored-by: Rida Hamadani --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-combinatorics new-contributor 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
57-6146
1 month ago
57-6147
57 days ago
71-35799
71 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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-set-theory 292/0 Mathlib.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/SetTheory/Cardinal/ENat.lean,Mathlib/SetTheory/Ordinal/Arithmetic.lean,Mathlib/SetTheory/Ordinal/Basic.lean,Mathlib/SetTheory/Ordinal/ENat.lean 6 9 ['github-actions', 'kckennylau', 'mathlib4-merge-conflict-bot'] alreadydone
assignee:alreadydone
57-6142
1 month ago
68-58364
68 days ago
71-18074
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-measure-probability 91/0 Mathlib.lean,Mathlib/MeasureTheory/Function/LInfty.lean 2 6 ['JonBannon', 'github-actions', 'j-loreaux', 'mathlib4-merge-conflict-bot'] nobody
57-6139
1 month ago
134-58036
134 days ago
4-6083
4 days
29411 llllvvuu
author:llllvvuu
feat(LinearAlgebra/Matrix/Rank): rank factorization The rank factorization derived from `Module.finBasis`. Co-authored-by: Aristotle Harmonic --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
57-6120
1 month ago
82-71897
82 days ago
46-47927
46 days
29425 pechersky
author:pechersky
feat(NumberTheory/Padics/Torsion): `HasEnoughRootsOfUnity ℤ_[p] (p - 1)` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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 merge-conflict awaiting-author t-ring-theory 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
57-6118
1 month ago
60-73072
60 days ago
44-22808
44 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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra large-import
label:t-algebra$
13/0 Mathlib/LinearAlgebra/Eigenspace/Minpoly.lean 1 5 ['github-actions', 'llllvvuu', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
57-6114
1 month ago
unknown
unknown
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! [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-order 31/0 Mathlib.lean,Mathlib/Order/UpperLower/WellFounded.lean 2 3 ['github-actions', 'mathlib4-merge-conflict-bot', 'plp127'] bryangingechen
assignee:bryangingechen
57-6112
1 month ago
115-74905
115 days ago
10-84761
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-data 35/0 Mathlib/Data/Multiset/Fintype.lean 1 9 ['Ruben-VandeVelde', 'github-actions', 'llllvvuu', 'mathlib4-merge-conflict-bot', 'vihdzp', 'wwylele'] pechersky
assignee:pechersky
57-6108
1 month ago
57-6109
57 days ago
69-16483
69 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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author help-wanted t-data 198/0 Mathlib.lean,Mathlib/Data/Nat/Choose/Wolstenholme.lean 2 4 ['github-actions', 'mathlib4-merge-conflict-bot', 'yury-harmonic'] nobody
57-5537
1 month ago
unknown
unknown
29720 javra
author:javra
feat(CategoryTheory): `TransportEnrichment` and `ForgetEnrichment` as 2-functors --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-category-theory 63/1 Mathlib/CategoryTheory/Enriched/Basic.lean,Mathlib/CategoryTheory/Enriched/EnrichedCat.lean 2 2 ['github-actions', 'mathlib4-merge-conflict-bot'] nobody
57-5530
1 month ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-topology FLT large-import 25/0 Mathlib/Topology/Algebra/ContinuousMonoidHom.lean 1 3 ['github-actions', 'grunweg', 'mathlib4-merge-conflict-bot'] nobody
57-5516
1 month ago
unknown
unknown
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) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-combinatorics new-contributor 476/0 Mathlib.lean,Mathlib/Combinatorics/Digraph/Maps.lean 2 2 ['github-actions', 'mathlib4-merge-conflict-bot'] awainverse
assignee:awainverse
57-5512
1 month ago
57-5513
57 days ago
54-81855
54 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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-measure-probability 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
57-5508
1 month ago
unknown
unknown
30001 vihdzp
author:vihdzp
feat: concept generated by set of objects/attributes --- - [ ] depends on: #29996 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR t-order 270/99 Mathlib/Order/Concept.lean 1 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
57-5502
1 month ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-analysis t-measure-probability 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
57-5499
1 month ago
78-2198
78 days ago
31-49299
31 days
30022 ADedecker
author:ADedecker
feat: theory of `IsRightUniformGroup` and `IsLeftUniformGroup` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-topology 799/150 Mathlib/Topology/Algebra/IsUniformGroup/Basic.lean,Mathlib/Topology/Algebra/IsUniformGroup/Defs.lean 2 7 ['github-actions', 'mathlib4-merge-conflict-bot'] nobody
57-5498
1 month ago
unknown
unknown
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`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-meta 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
57-5493
1 month ago
64-65290
64 days ago
23-34889
23 days
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR t-analysis 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
57-5489
1 month ago
unknown
unknown
30105 slashbade
author:slashbade
feat: add `reap` as internal tactic --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict new-contributor large-import t-meta 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
57-5484
1 month ago
unknown
unknown
30121 idontgetoutmuch
author:idontgetoutmuch
Principal fiber bundle core A structure capturing what it means to be a principal fibre bundle. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-differential-geometry new-contributor 227/0 Mathlib.lean,Mathlib/Geometry/Manifold/PrincipalFiberBundle/PrincipalGBundle.lean 2 6 ['github-actions', 'grunweg', 'mathlib4-merge-conflict-bot'] hrmacbeth
assignee:hrmacbeth
57-5479
1 month ago
79-65335
79 days ago
24-28967
24 days
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR new-contributor t-measure-probability 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
57-5343
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-ring-theory 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
57-5336
1 month ago
98-20
97 days ago
1-34346
1 day
30330 Bergschaf
author:Bergschaf
feat(Algebra/Group/Action/Equidecomp): Mathlib's definition of Equidecomposability is equivalent to the standart one using partitions --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra large-import
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
57-5335
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-ring-theory 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
57-5332
1 month ago
unknown
unknown
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]`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-data 41/0 Mathlib.lean,Mathlib/Data/FunLike/Graded.lean 2 2 ['github-actions', 'mathlib4-merge-conflict-bot'] nobody
57-5324
1 month ago
57-5325
57 days ago
40-71592
40 days
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
57-5320
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR t-data 78/0 Mathlib.lean,Mathlib/Data/FunLike/Graded.lean 2 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
57-5319
1 month ago
97-74442
97 days ago
0-1126
18 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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author blocked-by-other-PR t-meta 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
57-5316
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
57-5314
1 month ago
97-58071
97 days ago
0-2352
39 minutes
30392 urkud
author:urkud
feat: define pullback quotient maps --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-topology 287/0 Mathlib.lean,Mathlib/Topology/ClusterPt.lean,Mathlib/Topology/Maps/PullbackQuotient.lean 3 2 ['github-actions', 'mathlib4-merge-conflict-bot'] nobody
57-5311
1 month ago
unknown
unknown
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) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-ring-theory 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
57-5309
1 month ago
78-62716
78 days ago
16-68115
16 days
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 := ℤ`.) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-category-theory 134/0 Mathlib.lean,Mathlib/CategoryTheory/Linear/Linearization.lean 2 4 ['github-actions', 'joelriou', 'kim-em', 'mathlib4-merge-conflict-bot'] nobody
57-5003
1 month ago
78-33021
78 days ago
2-32784
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-measure-probability 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
57-4982
1 month ago
unknown
unknown
31102 JOSHCLUNE
author:JOSHCLUNE
Require LeanHammer Experimenting with adding LeanHammer as a mathlib dependency --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict new-contributor 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
57-4969
1 month ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-meta 151/11 Mathlib/Tactic/Check.lean,MathlibTest/Check.lean 2 12 ['github-actions', 'grunweg', 'mathlib4-merge-conflict-bot', 'thorimur'] thorimur
assignee:thorimur
57-4944
1 month ago
61-42482
61 days ago
11-39070
11 days
31314 hrmacbeth
author:hrmacbeth
feat: linters for recommended `field_simp` style --- - [x] depends on: #31472 - [x] depends on: #31483 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-linter awaiting-CI 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
57-4803
1 month ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-differential-geometry 591/0 Mathlib.lean,Mathlib/Geometry/Manifold/HasSmoothBoundary.lean 2 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
57-4577
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-algebra new-contributor merge-conflict awaiting-author
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
57-2344
1 month ago
unknown
unknown
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 -/ ``` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-meta 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
57-533
1 month ago
57-534
57 days ago
11-59965
11 days
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-differential-geometry blocked-by-other-PR merge-conflict t-meta 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
57-242
1 month ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-analysis 51/0 Mathlib.lean,Mathlib/Analysis/Analytic/Dslope.lean 2 26 ['github-actions', 'grunweg', 'maksym-radziwill', 'mathlib4-merge-conflict-bot'] nobody
57-237
1 month ago
62-41553
62 days ago
0-2120
35 minutes
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-category-theory 397/0 Mathlib.lean,Mathlib/CategoryTheory/Category/Quiv/AsOfFunctor.lean 2 13 ['github-actions', 'joelriou', 'mathlib4-merge-conflict-bot', 'robertmaxton42'] nobody
57-194
1 month ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-measure-probability 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
56-81808
1 month ago
unknown
unknown
21915 YaelDillies
author:YaelDillies
feat: simproc for `Int.divisorsAntidiag` Co-authored-by: Paul Lezeau --- - [x] depends on: #21912 - [x] depends on: #21991 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-meta 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
56-80677
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-analysis 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
56-80621
1 month ago
unknown
unknown
19475 YaelDillies
author:YaelDillies
feat: group markings From LeanCamCombi --- - [ ] depends on: #21342 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-algebra blocked-by-other-PR
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
56-80497
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-analysis 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
56-80333
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-differential-geometry 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
56-76585
1 month ago
57-70908
57 days ago
6-2726
6 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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-differential-geometry 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
56-72667
1 month ago
unknown
unknown
31338 grunweg
author:grunweg
chore: move Pretrivialization, Trivialization to the Bundle namespace As suggested in #30083. --- - [ ] depends on: #30083 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-differential-geometry 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
56-68119
1 month ago
69-30832
69 days ago
0-1063
17 minutes
31339 grunweg
author:grunweg
Movelemma --- - [ ] depends on: #31338 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
56-68117
1 month ago
69-30833
69 days ago
0-1120
18 minutes
31590 SuccessMoses
author:SuccessMoses
chore: tag `commutatorElement_def` with `simp` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-algebra new-contributor
label:t-algebra$
1/0 Mathlib/Algebra/Group/Commutator.lean 1 2 ['github-actions', 'grunweg'] nobody
56-66619
1 month ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
56-66545
1 month ago
62-78859
62 days ago
0-5
5 seconds
25802 dagurtomas
author:dagurtomas
feat(AlgebraicTopology): anodyne morphisms of simplicial sets --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) --- *This PR continues the work from #20201.* *Original PR: https://github.com/leanprover-community/mathlib4/pull/20201* WIP t-topology 145/0 Mathlib/AlgebraicTopology/Anodyne.lean,Mathlib/AlgebraicTopology/KanFibration.lean,Mathlib/CategoryTheory/MorphismProperty/WeakSaturation.lean 3 2 ['github-actions', 'mathlib4-merge-conflict-bot'] nobody
56-66526
1 month ago
unknown
unknown
6268 eric-wieser
author:eric-wieser
fix: fixups to #3838 This is an attempt to make #3838 universe polymorphic --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
56-65870
1 month ago
unknown
unknown
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) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP help-wanted CI 114/0 .github/workflows/mk_windows_bundle.yml,scripts/windowsBundle.bat 2 0 [] nobody
56-65862
1 month ago
unknown
unknown
6993 jjaassoonn
author:jjaassoonn
feat: lemmas about `AddMonoidAlgebra.{divOf, modOf}` --- - [x] depends on: #7582 - [x] depends on: #8975 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra
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
56-65857
1 month ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
56-65825
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-ring-theory 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
56-65810
1 month ago
unknown
unknown
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.) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-algebra
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
56-65804
1 month ago
unknown
unknown
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) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-algebra RFC
label:t-algebra$
86/0 Mathlib.lean,Mathlib/LinearAlgebra/LinearProgramming.lean 2 10 ['eric-wieser', 'madvorak', 'mathlib4-merge-conflict-bot', 'riccardobrasca'] nobody
56-65798
1 month ago
unknown
unknown
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) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-algebra RFC
label:t-algebra$
83/0 Mathlib.lean,Mathlib/LinearAlgebra/LinearProgramming.lean 2 8 ['eric-wieser', 'madvorak', 'mathlib4-merge-conflict-bot', 'riccardobrasca'] nobody
56-65791
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-category-theory 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
56-65768
1 month ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-algebraic-topology new-contributor 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
56-65760
1 month ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) please-adopt merge-conflict t-topology awaiting-zulip 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
56-65726
1 month ago
unknown
unknown
12087 JADekker
author:JADekker
feat: complete API for K-Lindelöf spaces --- - [ ] depends on: #11800 (which is now awaiting a design decision) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) please-adopt merge-conflict t-topology 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
56-65719
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-algebra t-order
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 3 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
56-65704
1 month 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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) please-adopt merge-conflict awaiting-author t-measure-probability 503/0 Mathlib.lean,Mathlib/MeasureTheory/Measure/Tight.lean 2 34 ['EtienneC30', 'JADekker', 'github-actions', 'sgouezel'] nobody
56-65699
1 month ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology awaiting-CI 75/0 Mathlib/Order/Filter/Cocardinal.lean 1 0 [] nobody
56-65695
1 month ago
unknown
unknown
14426 adomani
author:adomani
feat: `#min_imps` command (development branch) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
56-65666
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) please-adopt WIP workshop-AIM-AG-2024 merge-conflict t-algebraic-geometry 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
56-65655
1 month ago
unknown
unknown
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). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-algebra
label:t-algebra$
111/0 Mathlib.lean,Mathlib/LinearAlgebra/RootSystem/Separation.lean 2 1 ['github-actions'] nobody
56-65620
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP blocked-by-other-PR t-category-theory large-import merge-conflict t-algebraic-geometry 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 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
56-65613
1 month ago
unknown
unknown
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) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-algebra new-contributor
label:t-algebra$
91/0 Mathlib.lean,Mathlib/GroupTheory/SpecificGroups/BraidGroup/Basic.lean 2 22 ['github-actions', 'hannahfechtner', 'jcommelin', 'joelriou'] nobody
56-65607
1 month ago
unknown
unknown
18784 erdOne
author:erdOne
feat(AlgebraicGeometry): use `addMorphismPropertyInstances` --- - [ ] depends on: #18785 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebraic-geometry 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
56-65598
1 month ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-algebra
label:t-algebra$
38/0 Mathlib/GroupTheory/Congruence/Defs.lean 1 8 ['github-actions', 'hannahfechtner', 'kbuzzard', 'riccardobrasca'] nobody
56-65593
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP blocked-by-other-PR 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
56-65583
1 month ago
unknown
unknown
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.  --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP new-contributor t-meta 34/4 Mathlib/Tactic/Simps/Basic.lean 1 11 ['FrederickPu', 'YaelDillies', 'fpvandoorn', 'github-actions', 'leanprover-community-bot-assistant'] nobody
56-65544
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-category-theory new-contributor merge-conflict awaiting-author 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
56-65517
1 month ago
unknown
unknown
22805 ScottCarnahan
author:ScottCarnahan
feat(FieldTheory/Finite): fixed points of Frobenius automorphism This PR identifies the prime field with the fixed points of frobenius. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-algebra
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
56-65505
1 month ago
unknown
unknown
23772 SEU-Prime
author:SEU-Prime
feat: Amice equivalence i built amice equiv [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-number-theory 283/0 Mathlib/NumberTheory/Padics/Amice.lean 1 2 ['grunweg'] nobody
56-65486
1 month ago
unknown
unknown
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$. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-category-theory new-contributor 33/0 Mathlib/CategoryTheory/Limits/Types/Colimits.lean 1 5 ['github-actions', 'joelriou', 'leanprover-community-bot-assistant', 'robertmaxton42'] nobody
56-65400
1 month ago
unknown
unknown
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`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-data 31/0 Mathlib/Data/ULift.lean 1 23 ['eric-wieser', 'github-actions', 'grunweg', 'robertmaxton42'] nobody
56-65396
1 month ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-order 141/0 Mathlib.lean,Mathlib/Data/Prod/RevLex.lean 2 5 ['ScottCarnahan', 'YaelDillies', 'github-actions', 'mathlib4-merge-conflict-bot'] YaelDillies
assignee:YaelDillies
56-65386
1 month ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-order 35/0 Mathlib/RingTheory/HahnSeries/Basic.lean 1 2 ['github-actions', 'mathlib4-merge-conflict-bot'] nobody
56-65380
1 month ago
unknown
unknown
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₂`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-algebra
label:t-algebra$
28/0 Mathlib/Algebra/Module/Equiv/Basic.lean 1 1 ['github-actions'] nobody
56-65373
1 month ago
unknown
unknown
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₂`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-algebra
label:t-algebra$
21/0 Mathlib/Algebra/Module/Equiv/Defs.lean 1 1 ['github-actions'] nobody
56-65363
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) --- *This PR continues the work from #24102.* *Original PR: https://github.com/leanprover-community/mathlib4/pull/24102* merge-conflict WIP t-ring-theory 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
56-65345
1 month ago
72-82797
72 days ago
80-42499
80 days
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) --- *This PR continues the work from #24542.* *Original PR: https://github.com/leanprover-community/mathlib4/pull/24542* merge-conflict t-topology blocked-by-other-PR 716/65 Mathlib.lean,Mathlib/Data/Set/Accumulate.lean,Mathlib/Data/Set/Dissipate.lean,Mathlib/Data/Set/Prod.lean,Mathlib/MeasureTheory/Constructions/Cylinders.lean,Mathlib/MeasureTheory/Constructions/ProjectiveFamilyContent.lean,Mathlib/MeasureTheory/PiSystem.lean,Mathlib/Topology/Compactness/CompactSystem.lean 8 4 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
56-65322
1 month ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-data new-contributor 15/0 Mathlib/Data/Finset/Card.lean,Mathlib/Data/Set/Finite/Basic.lean 2 5 ['Ruben-VandeVelde', 'github-actions'] nobody
56-65311
1 month ago
198-2134
198 days ago
13-83428
13 days
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) --- *This PR continues the work from #24543.* *Original PR: https://github.com/leanprover-community/mathlib4/pull/24543* merge-conflict t-topology blocked-by-other-PR 996/66 Mathlib.lean,Mathlib/Data/Set/Accumulate.lean,Mathlib/Data/Set/Dissipate.lean,Mathlib/Data/Set/Prod.lean,Mathlib/MeasureTheory/Constructions/Cylinders.lean,Mathlib/MeasureTheory/Constructions/ProjectiveFamilyContent.lean,Mathlib/MeasureTheory/PiSystem.lean,Mathlib/Topology/Compactness/CompactSystem.lean 8 4 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
56-65302
1 month ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-algebra
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
56-65219
1 month ago
202-34889
202 days ago
0-15367
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-combinatorics 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
56-65194
1 month ago
57-6624
57 days ago
137-24962
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-set-theory 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
56-65172
1 month ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-analysis new-contributor 50/2 Mathlib/Analysis/Calculus/Deriv/Star.lean 1 15 ['emo916math', 'github-actions', 'j-loreaux', 'kckennylau'] j-loreaux
assignee:j-loreaux
56-65166
1 month ago
159-64914
159 days ago
31-69534
31 days
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-category-theory 1372/19 Mathlib.lean,Mathlib/CategoryTheory/Functor/KanExtension/Basic.lean,Mathlib/CategoryTheory/Monoidal/DayConvolution.lean,Mathlib/CategoryTheory/Monoidal/DayConvolution/DayFunctor.lean 4 5 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
56-65160
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-algebra
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
56-65138
1 month ago
148-62159
148 days ago
7-8492
7 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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-algebra
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
56-65114
1 month ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-data new-contributor 22/0 Mathlib/Data/Rat/Lemmas.lean 1 33 ['github-actions', 'kim-em', 'mathlib-bors', 'pechersky', 'sinianluoye', 'themathqueen'] pechersky
assignee:pechersky
56-65083
1 month ago
88-2277
88 days ago
74-50277
74 days
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 --> [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP new-contributor merge-conflict awaiting-author t-combinatorics 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
56-65062
1 month ago
unknown
unknown
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 :-( --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-algebra
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
56-65010
1 month ago
100-56533
100 days ago
40-64146
40 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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-algebra
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
56-64999
1 month ago
130-5784
130 days ago
5-4330
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` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-data 2/3 Mathlib/Data/Fin/Embedding.lean 1 2 ['github-actions', 'mathlib4-merge-conflict-bot'] nobody
56-64970
1 month ago
115-74869
115 days ago
18-35802
18 days
29514 grunweg
author:grunweg
feat(CI): use more strict mode --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP CI 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
56-64958
1 month ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-ring-theory new-contributor 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
56-64951
1 month ago
122-22281
122 days ago
1-40501
1 day
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR large-import 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
56-64885
1 month ago
unknown
unknown
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 blocked-by-other-PR t-category-theory new-contributor merge-conflict awaiting-author 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
56-64863
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP blocked-by-other-PR 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
56-64842
1 month ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-category-theory 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
56-64837
1 month ago
78-47001
78 days ago
2-38062
2 days
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR t-analysis new-contributor 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
56-64801
1 month ago
unknown
unknown
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. awaiting-author t-measure-probability new-contributor 13/0 Mathlib/MeasureTheory/PiSystem.lean 1 14 ['EtienneC30', 'KiringYJ', 'dagurtomas', 'github-actions', 'ocfnash'] RemyDegenne
assignee:RemyDegenne
56-51259
1 month ago
56-51259
56 days ago
135-34213
135 days
29409 Julian
author:Julian
feat(Mathlib/Analysis): deriv_eq_self and deriv_exp_iff --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-analysis 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
55-65224
1 month ago
113-56631
113 days ago
15-74499
15 days
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR t-meta 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
55-54406
1 month ago
64-60704
64 days ago
0-462
7 minutes
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
54-80936
1 month ago
58-79754
58 days ago
70-2909
70 days
29434 ntapiam
author:ntapiam
feat(NonAssoc/LieAdmissible): prove every ring/algebra is LieAdmissible -awaiting-author t-algebra new-contributor
label:t-algebra$
27/6 Mathlib/Algebra/NonAssoc/LieAdmissible/Defs.lean 1 2 ['github-actions', 'mathlib4-merge-conflict-bot'] nobody
54-49569
1 month ago
unknown
unknown
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-differential-geometry blocked-by-other-PR 390/11 Mathlib.lean,Mathlib/Analysis/InnerProductSpace/GramSchmidtOrtho.lean,Mathlib/Geometry/Manifold/VectorBundle/GramSchmidtOrtho.lean,scripts/noshake.json 4 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
54-43948
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-differential-geometry blocked-by-other-PR 927/11 Mathlib.lean,Mathlib/Analysis/InnerProductSpace/GramSchmidtOrtho.lean,Mathlib/Geometry/Manifold/Elaborators.lean,Mathlib/Geometry/Manifold/Traces.lean,Mathlib/Geometry/Manifold/VectorBundle/GramSchmidtOrtho.lean,scripts/noshake.json 6 6 ['faenuccio', 'github-actions', 'grunweg', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
54-43944
1 month ago
unknown
unknown
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] --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP blocked-by-other-PR new-contributor awaiting-author t-analysis 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
54-570
1 month ago
unknown
unknown
28141 YaelDillies
author:YaelDillies
chore: deprecate `BialgHom.coe_toLinearMap` `BialgHom.toLinearMap` is a fake projection. From Toric --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-ring-theory awaiting-zulip toric 5/11 Mathlib/RingTheory/Bialgebra/Hom.lean 1 16 ['YaelDillies', 'erdOne', 'eric-wieser', 'github-actions'] alreadydone
assignee:alreadydone
53-75571
1 month ago
53-75571
53 days ago
100-70827
100 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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics new-contributor 209/0 Mathlib/Combinatorics/SetFamily/Lindstrom.lean 1 2 ['github-actions', 'mathlib4-merge-conflict-bot'] b-mehta
assignee:b-mehta
53-73408
1 month ago
57-5167
57 days ago
31-45300
31 days
31949 ADedecker
author:ADedecker
chore: prefer `Pi.single i 1 j` over `fun j => if i = j then 1 else 0` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
53-39757
1 month ago
53-39757
53 days ago
0-21788
6 hours
29499 chrisflav
author:chrisflav
feat(CategoryTheory/Sites): sheafification via hypercovers This is very much WIP, but I need a fresh cache. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-category-theory 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
52-79549
1 month ago
unknown
unknown
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* t-measure-probability brownian large-import 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
52-70403
1 month ago
117-79203
117 days ago
29-52417
29 days
29030 b-mehta
author:b-mehta
feat(Combinatorics): prove the Rado selection lemma Prove the Rado selection lemma, a generic result useful to prove a variety of compactness results in combinatorics. This generalises Konig's infinity lemma, and the de Bruijn-Erdos theorem, and allows the former to be conveniently stated in the language of sets rather than categories. This is a draft PR for now, since de Bruijn-Erdos should move out of this file. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics 131/0 Mathlib/Combinatorics/SimpleGraph/DeBruijnErdos.lean 1 1 ['github-actions'] nobody
52-55035
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology blocked-by-other-PR new-contributor 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
52-48080
1 month ago
unknown
unknown
31571 erdOne
author:erdOne
feat(RingTheory): existence of local algebra with given residue field --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-ring-theory 225/0 Mathlib.lean,Mathlib/RingTheory/LocalRing/SeparableResidueField.lean 2 7 ['chrisflav', 'github-actions', 'jcommelin', 'mathlib4-merge-conflict-bot'] chrisflav
assignee:chrisflav
52-45192
1 month ago
52-48649
52 days ago
9-71460
9 days
29517 pechersky
author:pechersky
feat(RingTheory/Torsion): torsion = union of roots of unity with additional API for Associates and rootsOfUnity sups --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) - [x] depends on: #29988 - [x] depends on: #29989 - [x] depends on: #29990 - [x] depends on: #29991 merge-conflict awaiting-author t-algebra
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
52-38016
1 month ago
72-45819
72 days ago
37-64557
37 days
31176 mcdoll
author:mcdoll
feat(Analysis): Taylor's theorem with the integral remainder --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
52-2657
1 month ago
52-2657
52 days ago
7-28097
7 days
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
51-83847
1 month ago
unknown
unknown
28933 artie2000
author:artie2000
chore(Data): correct definition for `single_apply` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
51-82524
1 month ago
unknown
unknown
24627 pechersky
author:pechersky
feat(Topology/Algebra/Valued): `IsLinearTopology 𝒪[K] K` and `𝒪[K] 𝒪[K]` as well as `IsLinearTopology ℤ_[p] ℤ_[p]` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) - [x] depends on: #26829 merge-conflict awaiting-author t-topology 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
51-78138
1 month ago
57-7134
57 days ago
16-36220
16 days
27756 grunweg
author:grunweg
feat: `Weak(Pseudo)EMetricSpace`, generalises `(Pseudo)EMetricSpace` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-topology carleson 142/36 Mathlib/Topology/EMetricSpace/Defs.lean,Mathlib/Topology/Instances/ENNReal/Lemmas.lean 2 2 ['github-actions', 'mathlib4-merge-conflict-bot'] nobody
51-62889
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-data 21/31 Mathlib/Data/Finsupp/Single.lean 1 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
51-52183
1 month ago
unknown
unknown
26975 Whysoserioushah
author:Whysoserioushah
feat: a norm_num extension for complex numbers co-authored-by : @thefundamentaltheor3m, @hrmacbeth --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
51-42488
1 month ago
70-44565
70 days ago
111-3153
111 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) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-ring-theory 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
51-39571
1 month ago
51-78027
51 days ago
4-23266
4 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). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
51-36405
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-topology 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
51-25527
1 month ago
unknown
unknown
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`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
51-8391
1 month ago
53-37476
53 days ago
13-3239
13 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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-linter CI 154/0 lakefile.lean,scripts/run_linter.lean 2 1 ['github-actions'] nobody
50-79263
1 month ago
50-75663
50 days ago
50-75483
50 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! --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) please-adopt WIP merge-conflict 320/146 Mathlib/Analysis/LocallyConvex/Bounded.lean,Mathlib/Analysis/Oscillation.lean,Mathlib/Geometry/Manifold/LocalInvariantProperties.lean,Mathlib/MeasureTheory/Measure/EverywherePos.lean,Mathlib/SetTheory/Ordinal/Topology.lean,Mathlib/Topology/Algebra/Group/Basic.lean,Mathlib/Topology/Algebra/Module/Basic.lean,Mathlib/Topology/Algebra/Monoid.lean,Mathlib/Topology/Bases.lean,Mathlib/Topology/Basic.lean,Mathlib/Topology/Category/TopCat/Basic.lean,Mathlib/Topology/Clopen.lean,Mathlib/Topology/CompactOpen.lean,Mathlib/Topology/Compactness/LocallyCompact.lean,Mathlib/Topology/Constructions.lean,Mathlib/Topology/ContinuousOn.lean,Mathlib/Topology/DenseEmbedding.lean,Mathlib/Topology/Gluing.lean,Mathlib/Topology/Homeomorph.lean,Mathlib/Topology/IndicatorConstPointwise.lean,Mathlib/Topology/Inseparable.lean,Mathlib/Topology/Irreducible.lean,Mathlib/Topology/IsLocalHomeomorph.lean,Mathlib/Topology/LocalAtTarget.lean,Mathlib/Topology/Maps/Basic.lean,Mathlib/Topology/MetricSpace/Isometry.lean,Mathlib/Topology/NoetherianSpace.lean,Mathlib/Topology/Order.lean,Mathlib/Topology/Order/LowerUpperTopology.lean,Mathlib/Topology/Partial.lean,Mathlib/Topology/PartialHomeomorph.lean,Mathlib/Topology/PartitionOfUnity.lean,Mathlib/Topology/QuasiSeparated.lean,Mathlib/Topology/Separation.lean,Mathlib/Topology/TietzeExtension.lean,Mathlib/Topology/UniformSpace/Ascoli.lean,Mathlib/Topology/UniformSpace/Basic.lean,Mathlib/Topology/UniformSpace/Cauchy.lean,Mathlib/Topology/UniformSpace/CompactConvergence.lean,Mathlib/Topology/UniformSpace/Completion.lean,Mathlib/Topology/UniformSpace/Equicontinuity.lean,Mathlib/Topology/UniformSpace/Matrix.lean,Mathlib/Topology/UniformSpace/Pi.lean,Mathlib/Topology/UnitInterval.lean,Mathlib/Topology/UrysohnsBounded.lean,Mathlib/Topology/UrysohnsLemma.lean,Mathlib/Topology/VectorBundle/Basic.lean,lakefile.lean,scripts/run_linter.lean 49 0 [] nobody
50-79171
1 month ago
unknown
unknown
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis new-contributor awaiting-author 64/5 Mathlib/Analysis/SpecialFunctions/Stirling.lean 1 15 ['FaffyWaffles', 'github-actions', 'j-loreaux', 'mathlib4-merge-conflict-bot', 'tb65536'] nobody
50-42744
1 month ago
50-42744
50 days ago
4-54198
4 days
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author large-import t-meta 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
50-24774
1 month ago
60-79360
60 days ago
48-74529
48 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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-differential-geometry blocked-by-other-PR merge-conflict 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 12 ['github-actions', 'grunweg', 'idontgetoutmuch', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
50-21383
1 month ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data new-contributor 23/0 Mathlib/Data/EReal/Operations.lean 1 4 ['JovanGerb', 'LLaurance', 'dobronx1325', 'github-actions'] nobody
50-21050
1 month ago
50-77362
50 days ago
6-21252
6 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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-meta 36/23 Mathlib/Tactic/Ring/Basic.lean 1 2 ['github-actions', 'mathlib4-merge-conflict-bot'] nobody
50-20222
1 month ago
unknown
unknown
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
50-17088
1 month ago
68-79400
68 days ago
9-65641
9 days
31920 thorimur
author:thorimur
test: `env_linter` for unused decidable instances --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
50-16836
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-differential-geometry blocked-by-other-PR t-meta 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
49-82255
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
49-77623
1 month ago
49-77624
49 days ago
69-35285
69 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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
49-72728
1 month ago
49-72728
49 days ago
64-793
64 days
26138 xroblot
author:xroblot
Development branch (2) --- WIP merge-conflict 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 16 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-merge-conflict-bot'] nobody
49-61704
1 month ago
unknown
unknown
29357 eric-wieser
author:eric-wieser
refactor: generalize IsSimpleRing to semirings --- - [ ] depends on: #26277 - [ ] depends on: #22954 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
49-61200
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR large-import 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
49-46030
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
49-36565
1 month ago
49-36566
49 days ago
0-545
9 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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author blocked-by-other-PR t-order 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
49-6710
1 month ago
188-60462
188 days ago
0-17391
4 hours
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`. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data awaiting-author awaiting-zulip 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
49-6248
1 month ago
49-6248
49 days ago
35-75966
35 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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-order
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
49-5243
1 month ago
57-6632
57 days ago
26-48268
26 days
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`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-data awaiting-author 53/48 Mathlib/Data/Nat/Prime/Defs.lean 1 3 ['digama0', 'github-actions', 'leanprover-community-bot-assistant'] nobody
49-4016
1 month ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-data merge-conflict 44/22 Mathlib/Data/Int/GCD.lean 1 6 ['astrainfinita', 'b-mehta', 'eric-wieser', 'github-actions', 'mathlib4-merge-conflict-bot', 'nomeata', 'urkud'] nobody
48-80946
1 month ago
unknown
unknown
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$. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis new-contributor awaiting-author 14/0 Mathlib/Analysis/Convolution.lean 1 3 ['github-actions', 'urkud'] nobody
48-7430
1 month ago
48-7430
48 days ago
0-81373
22 hours
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) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
47-77625
1 month ago
57-4966
57 days ago
18-30750
18 days
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP blocked-by-other-PR t-category-theory awaiting-CI large-import merge-conflict 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
47-63364
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
47-59879
1 month ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP awaiting-author t-category-theory merge-conflict 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
47-58211
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP FLT 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
47-55017
1 month ago
112-86118
112 days ago
0-1383
23 minutes
29933 smmercuri
author:smmercuri
chore: fix `def` naming isses in `Normed/Field/WithAbs.lean` --- - [x] depends on: #29932 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP merge-conflict 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
47-54489
1 month ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis t-measure-probability 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
47-53473
1 month ago
48-77592
48 days ago
6-12807
6 days
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 t-number-theory blocked-by-other-PR large-import merge-conflict FLT 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
47-50828
1 month ago
unknown
unknown
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. merge-conflict WIP t-differential-geometry blocked-by-other-PR 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
47-47195
1 month ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-analysis new-contributor 331/0 Mathlib/Analysis/Normed/Operator/SingularValues.lean 1 2 ['github-actions', 'nielsvoss'] nobody
47-44971
1 month ago
unknown
unknown
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 WIP t-topology t-analysis
label:t-algebra$
150/0 Mathlib/RingTheory/Perfectoid.lean 1 2 ['github-actions', 'jjdishere'] nobody
47-2854
1 month ago
unknown
unknown
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 WIP t-number-theory t-algebra t-topology
label:t-algebra$
439/0 Mathlib/Topology/Algebra/Krasner.lean 1 3 ['github-actions', 'jjdishere', 'mathlib4-merge-conflict-bot'] nobody
47-2816
1 month ago
unknown
unknown
26961 mariainesdff
author:mariainesdff
feat(RingTheory/PowerSeries/Substitution): add API Co-authored-by: @AntoineChambert-Loir --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-ring-theory 57/4 Mathlib/RingTheory/PowerSeries/Basic.lean,Mathlib/RingTheory/PowerSeries/Substitution.lean 2 22 ['Ruben-VandeVelde', 'erdOne', 'github-actions', 'mariainesdff', 'mathlib4-merge-conflict-bot', 'mattrobball'] mattrobball
assignee:mattrobball
44-75209
1 month ago
60-75026
60 days ago
105-24099
105 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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
44-72658
1 month ago
44-72658
44 days ago
0-62409
17 hours
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
44-67898
1 month ago
44-67898
44 days ago
15-71432
15 days
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author merge-conflict 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
44-35474
1 month ago
51-84726
51 days ago
6-67021
6 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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
44-31269
1 month ago
47-15804
47 days ago
47-15624
47 days
32124 SnirBroshi
author:SnirBroshi
feat(SimpleGraph/Walks/Operations): expand basic drop/take/reverse API --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics 44/0 Mathlib/Combinatorics/SimpleGraph/Walks/Operations.lean 1 1 ['github-actions'] awainverse
assignee:awainverse
44-31259
1 month ago
50-22777
50 days ago
50-22597
50 days
25816 sgouezel
author:sgouezel
chore: kill coercion from EquivLike to Equiv --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-logic 35/37 Mathlib/Logic/Equiv/Defs.lean 1 2 ['github-actions', 'leanprover-community-bot-assistant'] nobody
43-78565
1 month ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP RFC 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
43-78545
1 month ago
unknown
unknown
29435 sgouezel
author:sgouezel
WIP: typeclass experiment --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-algebra
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
43-78529
1 month ago
unknown
unknown
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 awaiting-author t-algebra new-contributor
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
43-62820
1 month ago
82-5827
82 days ago
35-25302
35 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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
43-60792
1 month ago
unknown
unknown
31950 callesonne
author:callesonne
feat(CategoryTheory/Product/Basic): make `Hom` into a 1-field structure This should help unification. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-category-theory merge-conflict 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
43-59927
1 month ago
unknown
unknown
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 awaiting-author t-algebra merge-conflict
label:t-algebra$
277/5 Mathlib.lean,Mathlib/Analysis/Normed/Module/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 31 ['eric-wieser', 'github-actions', 'joelriou', 'leanprover-community-bot-assistant', 'mathlib4-merge-conflict-bot', 'riccardobrasca'] mattrobball
assignee:mattrobball
43-57074
1 month ago
85-65297
85 days ago
83-62164
83 days
8224 Kha
author:Kha
chore: add `lean4checker` benchmark WIP merge-conflict 16/0 scripts/bench/temci-config.run.yml 1 4 ['Kha', 'grunweg', 'kim-em', 'leanprover-bot', 'mathlib4-merge-conflict-bot'] nobody
43-46201
1 month ago
unknown
unknown
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
43-45059
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis new-contributor 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
43-35614
1 month ago
unknown
unknown
29393 staroperator
author:staroperator
feat(SetTheory/ZFC): `card (V_ o) = preBeth o` --- - [x] depends on: #26544 - [x] depends on: #29351 - [x] depends on: #29365 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
43-31255
1 month ago
47-20682
47 days ago
47-20502
47 days
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
43-894
1 month ago
43-895
43 days ago
35-52008
35 days
27579 RemyDegenne
author:RemyDegenne
feat: risk of an estimator, DeGroot statistical information, total variation distance This is an overview PR and will be cut into several pieces. It contains definitions and properties of: - the risk and Bayes risk of an estimator, in general and then specialized to binary hypothesis testing - the DeGroot statistical information between two measures, as well as a generalization for a kernel on more than two outcomes - the total variation distance between measures, defined as a special case of the DeGroot statistical information Co-authored-by: Lorenzo Luccioli @LorenzoLuccioli From the TestingLowerBounds project --- - [x] depends on: #27583 - [x] depends on: #27584 - [x] depends on: #27585 - [x] depends on: #27586 - [x] depends on: #27587 - [x] depends on: #27591 - [x] depends on: #28081 - [x] depends on: #28082 - [x] depends on: #28117 - [x] depends on: #28341 - [x] depends on: #29137 - [x] depends on: #29143 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP large-import t-measure-probability 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
42-74443
1 month ago
unknown
unknown
30966 gasparattila
author:gasparattila
refactor: disable `simp` in `measurability` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
42-67673
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
42-44069
1 month 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) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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. awaiting-author t-topology 6/1 Mathlib/Topology/Algebra/Module/ModuleTopology.lean 1 9 ['github-actions', 'j-loreaux', 'kbuzzard', 'leanprover-bot', 'ocfnash'] ocfnash
assignee:ocfnash
41-71560
1 month ago
108-70214
108 days ago
25-1060
25 days
32436 thorimur
author:thorimur
feat: `unusedFactInType` linter --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-linter 55/3 Mathlib/Init.lean,Mathlib/Tactic/Linter/UnusedInstancesInType.lean 2 1 ['github-actions'] nobody
41-50146
1 month 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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP blocked-by-other-PR merge-conflict 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
41-44756
1 month ago
unknown
unknown
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). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-algebra RFC merge-conflict
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
41-40232
1 month ago
53-37381
53 days ago
9-5002
9 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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
41-21091
1 month ago
57-202
57 days ago
2-24540
2 days
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order awaiting-author merge-conflict 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
41-14509
1 month ago
44-75503
44 days ago
24-12813
24 days
32474 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. --- This PR continues #23214 which was delegated by @j-loreaux but I let it slip. Will re-bench and see the effect. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
6/0 Mathlib/Algebra/Module/LinearMap/Defs.lean 1 1 ['github-actions'] nobody
40-70540
1 month ago
unknown
unknown
31898 ntapiam
author:ntapiam
feat(LinearAlgebra/TensorAlgebra): implement HopfAlgebra for TensorAlgebra implementation of the natural Hopf algebra structure on the TensorAlgebra new-contributor t-ring-theory 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 64 ['YaelDillies', 'github-actions', 'kckennylau', 'ntapiam'] nobody
40-65807
1 month ago
53-32620
53 days ago
0-30128
8 hours
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-meta merge-conflict 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 7 ['JovanGerb', 'fpvandoorn', 'github-actions', 'mathlib4-merge-conflict-bot', 'thorimur'] thorimur
assignee:thorimur
40-63076
1 month ago
54-60581
54 days ago
7-68317
7 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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-meta 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 13 ['bryangingechen', 'dwrensha', 'github-actions', 'mathlib4-merge-conflict-bot', 'urkud', 'vasnesterov', 'yury-harmonic'] nobody
40-61342
1 month 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`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-meta 152/1 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/NormNum/IsSquare.lean,MathlibTest/norm_num_ext.lean 4 16 ['Rob23oba', 'dwrensha', 'github-actions', 'mathlib4-merge-conflict-bot', 'plp127', 'vasnesterov', 'yury-harmonic'] dwrensha
assignee:dwrensha
40-59873
1 month ago
59-68498
59 days ago
35-83439
35 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. t-combinatorics new-contributor awaiting-author merge-conflict 113/0 Mathlib.lean,Mathlib/Combinatorics/Enumerative/Polya.lean 2 8 ['IvanRenison', 'alreadydone', 'github-actions', 'mathlib4-merge-conflict-bot'] awainverse
assignee:awainverse
40-52569
1 month ago
49-9712
49 days ago
39-39956
39 days
31113 515801431
author:515801431
feat(Mathlib/Combinatorics/Enumerative/Polya.lean): Add additional theorem in `Polya.lean` --- - [ ] depends on: #30525 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics new-contributor blocked-by-other-PR merge-conflict 302/0 Mathlib.lean,Mathlib/Combinatorics/Enumerative/Polya.lean 2 4 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] b-mehta
assignee:b-mehta
40-52445
1 month ago
49-74871
49 days ago
16-74719
16 days
29000 JovanGerb
author:JovanGerb
feat(Tactic/Push): add basic tags and tests This PR adds basic `@[push]` tags, and expands the `push` test file. --- - [ ] depends on: #21965 - [ ] depends on: #30038 - [ ] depends on: #30039 - [ ] depends on: #30042 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
40-51531
1 month ago
109-28139
109 days ago
0-9867
2 hours
24441 MrSumato
author:MrSumato
feat(Data/List): add Lyndon-Schutzenberger theorem on list commutativity Add Lyndon-Schutzenberger theorem on list commutativity. Included definition for List.repeatSelf that returns list repeated n times. --- This is my first mathlib PR, so any comments are highly appreciated. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-data new-contributor 129/1 Mathlib.lean,Mathlib/Data/List/Commutativity.lean,Mathlib/Data/List/Defs.lean,Mathlib/Data/List/Lemmas.lean 4 38 ['MrSumato', 'github-actions', 'grunweg', 'madvorak', 'mathlib4-merge-conflict-bot', 'plp127'] grunweg
assignee:grunweg
40-48047
1 month ago
unknown
unknown
32125 SnirBroshi
author:SnirBroshi
feat(SimpleGraph/Walks/Subwalks): `p₁.IsSubwalk p₂ ↔ p₁.darts <:+: p₂.darts` and similar theorems --- - [ ] depends on: #32160 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics blocked-by-other-PR 87/3 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
40-43472
1 month ago
49-25808
49 days ago
0-80872
22 hours
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 - [x] depends on: #29596 - [x] depends on: #29597 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra awaiting-author large-import
label:t-algebra$
676/6 Mathlib.lean,Mathlib/GroupTheory/MonoidLocalization/Archimedean.lean,Mathlib/GroupTheory/MonoidLocalization/Basic.lean,Mathlib/GroupTheory/MonoidLocalization/Lemmas.lean,Mathlib/RingTheory/IsTensorProduct.lean,Mathlib/RingTheory/Localization/Additive.lean,Mathlib/RingTheory/Localization/Defs.lean,Mathlib/RingTheory/Localization/StrongRankCondition.lean 8 6 ['alreadydone', 'chrisflav', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] chrisflav
assignee:chrisflav
40-30167
1 month ago
131-69173
131 days ago
11-86370
11 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]`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-order merge-conflict 8/2 Mathlib/Order/SuccPred/Basic.lean 1 4 ['YaelDillies', 'github-actions', 'mathlib4-merge-conflict-bot', 'plp127', 'vihdzp'] bryangingechen
assignee:bryangingechen
40-27675
1 month ago
117-43383
117 days ago
44-7812
44 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)`. Currently this introduces a new function `Nat.binom`, but we could also modify `Nat.multinomial`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data 226/1 Mathlib/Data/Nat/Choose/Binomial.lean,Mathlib/Data/Nat/Choose/Multinomial.lean 2 1 ['github-actions'] nobody
40-5935
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory awaiting-author 135/2 Mathlib.lean,Mathlib/CategoryTheory/Bicategory/Basic.lean,Mathlib/CategoryTheory/Bicategory/InducedBicategory.lean,Mathlib/CategoryTheory/Bicategory/Subbicategory.lean 4 7 ['callesonne', 'github-actions', 'leanprover-radar', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'robin-carlier'] nobody
39-80063
1 month ago
40-65144
40 days ago
2-58918
2 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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-ring-theory awaiting-author 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 4 ['erdOne', 'github-actions'] erdOne
assignee:erdOne
39-76445
1 month ago
39-76445
39 days ago
4-61403
4 days
32473 mattrobball
author:mattrobball
chore(Kaehler.JacobiZariski): remove egregious local instance hack This code looks terrible and is no longer strictly necessary. Local timings give `lake build Mathlib/RingTheory/Kaehler/JacobiZariski.lean 39.77s user 1.07s system 263% cpu 15.482 total` after removal and `lake build Mathlib/RingTheory/Kaehler/JacobiZariski.lean 36.93s user 1.01s system 251% cpu 15.113 total` before the removal. So the preformance impact of removal is small. One could argue that keeping is a remainder that everything here needs to be seriously changed but the miminmal performance difference suggests that these local instances would be a red herring in that regard. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-ring-theory awaiting-author 0/4 Mathlib/RingTheory/Kaehler/JacobiZariski.lean 1 13 ['chrisflav', 'erdOne', 'github-actions', 'leanprover-radar', 'mattrobball'] nobody
39-71670
1 month ago
39-71670
39 days ago
0-85695
23 hours
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-linter large-import 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 15 ['Hagb', 'github-actions', 'grunweg', 'mathlib4-merge-conflict-bot'] nobody
39-27234
1 month ago
unknown
unknown
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 - [x] depends on: #18534 - [x] 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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-algebra blocked-by-other-PR merge-conflict t-algebraic-geometry
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 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
38-68907
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 - [x] depends on: #25971 - [x] depends on: #13539 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-category-theory 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 23 ['alreadydone', 'callesonne', 'chrisflav', 'github-actions', 'joelriou', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'yuma-mizuno'] nobody
38-68548
1 month ago
unknown
unknown
32245 erdOne
author:erdOne
feat(RingTheory): the `coassoc_simps` simp set From Toric Co-authored-by: Yaël Dillies --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-ring-theory toric 836/0 Mathlib.lean,Mathlib/RingTheory/Coalgebra/CoassocSimps.lean,Mathlib/RingTheory/Coalgebra/SimpAttr.lean,MathlibTest/RingTheory/CoassocSimps.lean 4 1 ['github-actions'] nobody
38-60610
1 month 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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta 703/0 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/WildcardLevel.lean,MathlibTest/WildcardLevel.lean 4 25 ['JovanGerb', 'adamtopaz', 'github-actions'] dwrensha
assignee:dwrensha
38-31261
1 month ago
40-48972
40 days ago
42-30056
42 days
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics new-contributor 391/0 Mathlib.lean,Mathlib/Combinatorics/DiHypergraph/Basic.lean 2 2 ['github-actions', 'mathlib4-merge-conflict-bot'] b-mehta
assignee:b-mehta
37-75484
1 month ago
57-5527
57 days ago
57-67557
57 days
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-dynamics new-contributor awaiting-author 114/6 Mathlib/Dynamics/Transitive.lean 1 6 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'sgouezel'] sgouezel
assignee:sgouezel
37-73280
1 month ago
37-73280
37 days ago
18-34491
18 days
30711 kim-em
author:kim-em
experiment: which `omega` can not be replaced with `grind`? 1/0 lakefile.lean 1 2 ['github-actions', 'mathlib4-merge-conflict-bot'] nobody
37-66353
1 month ago
unknown
unknown
30718 kim-em
author:kim-em
experiment: merge rewrites t-meta 1/0 lakefile.lean 1 3 ['github-actions', 'mathlib4-merge-conflict-bot'] nobody
37-66351
1 month ago
unknown
unknown
30720 kim-em
author:kim-em
experiment: merge with subsequent grind 1/0 lakefile.lean 1 2 ['github-actions', 'mathlib4-merge-conflict-bot'] nobody
37-66351
1 month ago
unknown
unknown
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra awaiting-author merge-conflict
label:t-algebra$
566/487 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/FreeAlgebra.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/Congruence/Hom.lean,Mathlib/RingTheory/DedekindDomain/Different.lean,Mathlib/RingTheory/Etale/Field.lean,Mathlib/RingTheory/Etale/StandardEtale.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 104 63 ['fpvandoorn', 'github-actions', 'jcommelin', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'leanprover-radar', 'mathlib4-merge-conflict-bot', 'themathqueen'] joelriou
assignee:joelriou
37-46621
1 month ago
49-70881
49 days ago
65-33942
65 days
32455 vihdzp
author:vihdzp
feat: order topologies of successor orders --- Co-authored by @j-loreaux [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology t-order 124/43 Mathlib.lean,Mathlib/Order/Cover.lean,Mathlib/SetTheory/Ordinal/Topology.lean,Mathlib/Topology/Order/SuccPred.lean 4 1 ['github-actions'] pechersky
assignee:pechersky
37-31260
1 month ago
41-15159
41 days ago
41-14979
41 days
32614 vihdzp
author:vihdzp
refactor: Typeclass for antitone inverses/negation There are a couple of types with antitone inverses or negation that don't otherwise adhere to the group axioms. Examples include `SignType` and `EReal` for negation, and `ENNReal` for inverses. The CGT repository also adds the type of games and the type of surreal cuts to the list for negation. To standardize the various corollaries of this condition, we introduce mix-ins `NegAntiClass` and `InvAntiClass`. Lemmas which formerly required `Group` are now proven under weaker assumptions like `DivisionMonoid` or even `InvolutiveInv`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
161/82 Mathlib/Algebra/Order/Group/Defs.lean,Mathlib/Algebra/Order/Group/OrderIso.lean,Mathlib/Algebra/Order/Group/Unbundled/Basic.lean 3 2 ['github-actions', 'jsm28'] nobody
37-24322
1 month ago
unknown
unknown
25871 eric-wieser
author:eric-wieser
refactor: generalize rank lemmas to semirings --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict
label:t-algebra$
18/8 Mathlib/LinearAlgebra/Dimension/Finite.lean 1 2 ['github-actions', 'mathlib4-merge-conflict-bot'] nobody
37-21329
1 month ago
unknown
unknown
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/361 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 18 ['eric-wieser', 'github-actions', 'kim-em', 'mathlib4-merge-conflict-bot'] nobody
37-13827
1 month ago
unknown
unknown
30119 Ruben-VandeVelde
author:Ruben-VandeVelde
feat: WithTop/Bot.mapD To replace Option.elim; working towards #27918 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-order merge-conflict 32/4 Mathlib/Order/Hom/WithTopBot.lean,Mathlib/Order/WithBot.lean 2 5 ['JovanGerb', 'YaelDillies', 'github-actions', 'mathlib4-merge-conflict-bot'] YaelDillies
assignee:YaelDillies
37-13458
1 month ago
93-1550
93 days ago
12-88
12 days
32328 ADedecker
author:ADedecker
feat: template for distributions and their API --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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 4 ['github-actions', 'mathlib4-merge-conflict-bot'] nobody
36-43592
1 month ago
unknown
unknown
32458 vihdzp
author:vihdzp
feat: order isomorphisms preserve successor/predecessor limits Co-authored-by: Aaron Liu --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order awaiting-author 31/1 Mathlib/Order/SuccPred/Limit.lean 1 2 ['YaelDillies', 'github-actions'] YaelDillies
assignee:YaelDillies
36-8500
1 month ago
38-77471
38 days ago
2-15488
2 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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics new-contributor merge-conflict 375/0 Mathlib.lean,Mathlib/Combinatorics/Hypergraph/Basic.lean 2 54 ['b-mehta', 'espottesmith', 'github-actions', 'jt496', 'lauramonk', 'mathlib4-merge-conflict-bot'] b-mehta
assignee:b-mehta
36-6493
1 month ago
57-6283
57 days ago
76-50008
76 days
24000 YaelDillies
author:YaelDillies
feat: correspondence between affine group schemes and Hopf algebras 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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-algebraic-geometry toric FLT 127/0 Mathlib/AlgebraicGeometry/GroupScheme/HopfAffine.lean 1 3 ['YaelDillies', 'github-actions', 'kbuzzard'] nobody
36-2200
1 month ago
unknown
unknown
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 - [x] 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) - [x] 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.) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-differential-geometry blocked-by-other-PR 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
35-73437
1 month ago
unknown
unknown
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. --- - [ ] depends on: #32578 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-category-theory WIP 58/0 Mathlib/CategoryTheory/Sites/Sheaf.lean 1 5 ['chrisflav', 'github-actions', 'joelriou', 'mathlib4-dependent-issues-bot'] nobody
35-60292
1 month ago
207-709
207 days ago
1-59018
1 day
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. --- - [x] depends on: #10653 - [x] depends on: #10994 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP modifies-tactic-syntax t-meta 392/124 Mathlib/Tactic/TFAE.lean,scripts/noshake.json,test/tfae.lean 3 3 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
35-53684
1 month ago
unknown
unknown
30668 astrainfinita
author:astrainfinita
feat: `QuotType` This typeclass is primarily for use by type synonyms of `Quot` and `Quotient`. Using `QuotType` 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. [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 RFC t-data awaiting-zulip 629/0 Mathlib.lean,Mathlib/Data/QuotType.lean,MathlibTest/QuotType.lean 3 20 ['YaelDillies', 'astrainfinita', 'github-actions', 'mathlib4-merge-conflict-bot', 'plp127', 'vihdzp'] nobody
35-47572
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-euclidean-geometry blocked-by-other-PR 169/0 Mathlib/Analysis/Convex/Side.lean,Mathlib/Geometry/Euclidean/Incenter.lean 2 4 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
35-41639
1 month ago
45-62390
45 days ago
0-2574
42 minutes
32556 vihdzp
author:vihdzp
doc: fix URL in docs `doc-gen` splits the URL at every comma, so we replace them with the ASCII escape %2C instead. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) documentation awaiting-author 1/1 Counterexamples/EulerSumOfPowers.lean 1 3 ['eric-wieser', 'github-actions', 'ocfnash'] nobody
35-41590
1 month ago
37-85141
37 days ago
0-47028
13 hours
32706 CoolRmal
author:CoolRmal
feat: a set is Gdelta iff it is completely metrizable This PR proves that 1. A Gdelta subset of a completely metrizable space is completely metrizable. 2. We prove that under certain conditions we can always extends a continuous function on a set A to a Gdelta set. We then use this lemma to prove that if `A` is a completely metrizable subset in a metric space `M`, then `A` is Gdelta. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology 29/0 Mathlib/Topology/Metrizable/CompletelyMetrizable.lean 1 1 ['github-actions'] nobody
35-38316
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP blocked-by-other-PR t-category-theory merge-conflict 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 7 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
35-112
1 month ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order awaiting-author merge-conflict 22/0 Mathlib/Order/Defs/PartialOrder.lean 1 7 ['Vierkantor', 'github-actions', 'mathlib4-merge-conflict-bot', 'plp127'] Vierkantor
assignee:Vierkantor
34-85795
1 month ago
50-82266
50 days ago
19-72878
19 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`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-euclidean-geometry merge-conflict 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 13 ['JovanGerb', 'github-actions', 'jsm28', 'mathlib4-merge-conflict-bot'] jsm28
assignee:jsm28
34-85793
1 month ago
40-67651
40 days ago
41-522
41 days
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 --- - [ ] depends on: #32725 - [x] depends on: #32423 - [x] depends on: #32424 - [x] depends on: #30168 - [x] depends on: #30160 - [x] depends on: #29881 - [x] depends on: #29854 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-category-theory blocked-by-other-PR 292/0 Mathlib.lean,Mathlib/CategoryTheory/Limits/Types/Limits.lean,Mathlib/CategoryTheory/MorphismProperty/Basic.lean,Mathlib/CategoryTheory/MorphismProperty/IsSmall.lean,Mathlib/CategoryTheory/ObjectProperty/FunctorCategory/Presheaf.lean,Mathlib/CategoryTheory/ObjectProperty/Local.lean,Mathlib/CategoryTheory/Presentable/Continuous.lean 7 9 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
34-78810
1 month ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-analysis sphere-packing 199/0 Mathlib/Analysis/Complex/CauchyIntegral.lean 1 3 ['github-actions', 'mathlib4-merge-conflict-bot', 'wwylele'] nobody
34-70949
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-number-theory blocked-by-other-PR t-algebraic-geometry merge-conflict
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 4 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
34-68081
1 month ago
unknown
unknown
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 ``` --- - [x] depends on: #6227 for the `NoZeroDivisors` instance on `AddMonoidAlgebra`s [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-algebra
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 6 ['SnirBroshi', 'YaelDillies', 'adomani', 'eric-wieser', 'leanprover-community-mathlib4-bot'] nobody
34-67207
1 month ago
unknown
unknown
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). --- - [x] depends on: #31506 For full disclosure, most of the lemma statements in `Lemmas.lean` were generated by an LLM. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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 14 ['FLDutchmann', 'Vierkantor', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] Vierkantor
assignee:Vierkantor
34-50006
1 month ago
41-63012
41 days ago
9-5936
9 days
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`. --- - [x] depends on: #28793 - [ ] depends on: #28796 - [x] depends on: #28853 (for simplicity) - [ ] depends on: #28905 history bifurcates here: merge that PR first, then rebase this one [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-differential-geometry blocked-by-other-PR 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 5 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'peabrainiac'] nobody
34-34297
1 month ago
unknown
unknown
32609 PrParadoxy
author:PrParadoxy
feat(LinearAlgebra/PiTensorProduct): Relation between nested tensor products and tensor products indexed by dependent sums Product tensors in `⨂ j : (Σ i, β i), s j.fst j.snd` can be mapped to product tensors in `⨂ i, ⨂ b : β i, s i b`. If the outer index type is finite, the two types are equivalent. This allows the definition of endomorphisms on PiTensorProducts by specifying them on disjoint subsets of the index set. Such constructions are common e.g. in quantum circuits, quantum cellular automata, and renormalization procedures. --- WIP. This PR contains two "requests for comments". Essentially: * Is a single complex-to-define linear equivalence preferable over several less complex ones, which might however be of limited interest by themselves? * Which trade-offs are appropriate to make things computable? - [ ] depends on: #32608 - [ ] depends on: #32600 - [x] depends on: #32598 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor blocked-by-other-PR 683/0 Mathlib.lean,Mathlib/Data/Sigma/Basic.lean,Mathlib/LinearAlgebra/Multilinear/Basic.lean,Mathlib/LinearAlgebra/PiTensorProduct/Nested.lean,Mathlib/LinearAlgebra/PiTensorProduct/Set.lean 5 4 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
34-32413
1 month ago
37-43788
37 days ago
0-614
10 minutes
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-measure-probability new-contributor awaiting-author merge-conflict 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 7 ['github-actions', 'jcommelin', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'zhuyizheng'] sgouezel
assignee:sgouezel
34-13548
1 month ago
49-64644
49 days ago
1-22579
1 day
30666 erdOne
author:erdOne
feat(NumberTheory): every number field has a ramified prime --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-number-theory awaiting-author t-algebra merge-conflict
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 23 ['erdOne', 'github-actions', 'jcommelin', 'mathlib4-merge-conflict-bot', 'tb65536', 'xroblot'] jcommelin
assignee:jcommelin
34-12624
1 month ago
67-27521
67 days ago
13-60954
13 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 merge-conflict 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 5 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
34-12623
1 month ago
84-11942
84 days ago
0-1475
24 minutes
26950 alreadydone
author:alreadydone
Primitives of holomorphic functions and path integral --- - [ ] depends on: #31925 - [x] depends on: #24983 - [x] depends on: #22771 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP merge-conflict t-topology t-analysis blocked-by-other-PR 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 3 ['alreadydone', 'grunweg', 'mathlib4-dependent-issues-bot'] nobody
33-82988
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
33-67964
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
33-67963
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
33-67960
1 month ago
unknown
unknown
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 - [x] depends on: #30236 - [x] depends on: #30202 - [x] depends on: #30201 - [x] depends on: #30199 - [x] depends on: #30198 - [x] depends on: #30197 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR merge-conflict 463/18 Mathlib/Analysis/Distribution/ContDiffMapSupportedIn.lean 1 5 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
33-67959
1 month ago
unknown
unknown
32799 fpvandoorn
author:fpvandoorn
feat: add extra trace message to positivity * It's hard to follow what `positivity` is doing, even with the tracing on * This PR improves the situation a little bit by displaying a message after every positivity extension. * Could be potentially improved further by storing the names of positivity extensions in `PositivityExt`, but this is a simple change in the meantime --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta 1/0 Mathlib/Tactic/Positivity/Core.lean 1 1 ['github-actions'] nobody
33-63184
1 month ago
unknown
unknown
32798 fpvandoorn
author:fpvandoorn
perf: don't run positivityCanon if you already know nonnegative --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta 11/3 Mathlib/Tactic/Positivity/Core.lean 1 3 ['fpvandoorn', 'github-actions', 'leanprover-radar'] nobody
33-57079
1 month ago
unknown
unknown
32827 erdOne
author:erdOne
perf: `@[simp high]` on `*Hom.map_add` lemmas --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
10/0 Mathlib/Algebra/Module/Equiv/Defs.lean,Mathlib/Algebra/Module/LinearMap/Defs.lean,Mathlib/Algebra/Ring/Equiv.lean,Mathlib/Algebra/Ring/Hom/Defs.lean 4 3 ['erdOne', 'github-actions', 'leanprover-radar'] nobody
33-21885
1 month ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-topology 124/0 Mathlib/Analysis/Normed/Group/Basic.lean,Mathlib/Topology/MetricSpace/Basic.lean,Mathlib/Topology/MetricSpace/Pseudo/Constructions.lean 3 13 ['github-actions', 'kckennylau', 'mathlib4-merge-conflict-bot', 'pechersky', 'plp127'] urkud
assignee:urkud
32-31340
1 month ago
54-67949
54 days ago
113-59066
113 days
32552 ksenono
author:ksenono
feat(SetTheory/Cardinal): helpers for Konig's theorem --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-set-theory new-contributor 70/0 Mathlib/SetTheory/Cardinal/Arithmetic.lean,Mathlib/SetTheory/Cardinal/Basic.lean 2 33 ['SnirBroshi', 'b-mehta', 'github-actions', 'ksenono', 'staroperator', 'vihdzp'] b-mehta
assignee:b-mehta
32-15389
1 month ago
32-36797
32 days ago
37-79310
37 days
32869 felixpernegger
author:felixpernegger
feat(RingTheory): lemmas around ```Ring.choose``` Various small lemmas around Ring.choose. In particular this should cover all statements from .Data.Nat.Choose.Basic which have a meaningful generalization to arbitrary rings. new-contributor t-ring-theory 170/0 Mathlib/RingTheory/Binomial.lean,Mathlib/RingTheory/Polynomial/Pochhammer.lean 2 1 ['github-actions'] nobody
32-1745
1 month 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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) brownian t-measure-probability blocked-by-other-PR merge-conflict 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 5 ['EtienneC30', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
31-82804
1 month ago
44-40831
44 days ago
0-143
2 minutes
32704 euprunin
author:euprunin
chore: remove use of `erw` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-topology t-category-theory t-measure-probability 10/11 Mathlib/AlgebraicTopology/DoldKan/Homotopies.lean,Mathlib/CategoryTheory/Preadditive/AdditiveFunctor.lean,Mathlib/Topology/Homotopy/Product.lean 3 19 ['MichaelStollBayreuth', 'bryangingechen', 'euprunin', 'github-actions', 'grunweg', 'leanprover-radar'] MichaelStollBayreuth
assignee:MichaelStollBayreuth
31-67828
1 month ago
31-80082
31 days ago
3-17574
3 days
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-measure-probability new-contributor awaiting-author 21/0 Mathlib/Probability/Moments/Basic.lean 1 5 ['DavidLedvinka', 'github-actions'] RemyDegenne
assignee:RemyDegenne
31-65386
1 month ago
31-65386
31 days ago
21-30654
21 days
32600 PrParadoxy
author:PrParadoxy
feat(LinearAlgebra/Multilinear): composition of multilinear maps The composition of a multilinear map with a family of multilinear maps is a multilinear map indexed by a dependent sum. The result reduces to a lemma about the interaction of function application, `Sigma.curry`, and `Function.update`. This variant of `Function.apply_update` is included as `Sigma.apply_curry_update`. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor 40/0 Mathlib/Data/Sigma/Basic.lean,Mathlib/LinearAlgebra/Multilinear/Basic.lean 2 4 ['github-actions', 'goliath-klein', 'kbuzzard'] dwrensha
assignee:dwrensha
31-60260
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra blocked-by-other-PR large-import
label:t-algebra$
1234/17 Mathlib.lean,Mathlib/Algebra/BigOperators/Finprod.lean,Mathlib/Algebra/MvPolynomial/Equiv.lean,Mathlib/Algebra/MvPolynomial/RestrictedValue.lean,Mathlib/Algebra/Vertex/HVertexOperator.lean,Mathlib/Algebra/Vertex/VertexOperator.lean,Mathlib/RingTheory/Binomial.lean,Mathlib/RingTheory/HahnSeries/Addition.lean,Mathlib/RingTheory/HahnSeries/Binomial.lean,Mathlib/RingTheory/HahnSeries/HEval.lean,Mathlib/RingTheory/HahnSeries/Multiplication.lean,Mathlib/RingTheory/HahnSeries/Summable.lean,Mathlib/RingTheory/Polynomial/Pochhammer.lean 13 4 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
31-59751
1 month ago
118-68134
118 days ago
0-11779
3 hours
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 - [x] depends on: #30921 - [x] depends on: #32234 - [x] depends on: #32249 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) brownian t-measure-probability blocked-by-other-PR merge-conflict 725/1 Mathlib.lean,Mathlib/Probability/Distributions/Gaussian/Basic.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 6 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
31-48645
1 month ago
unknown
unknown
31766 SuccessMoses
author:SuccessMoses
feat(Topology/EMetricSpace): continuity of arc length fixes half of #31751 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-topology awaiting-author 396/0 Mathlib.lean,Mathlib/Topology/EMetricSpace/ArcLength.lean,Mathlib/Topology/EMetricSpace/BoundedVariation.lean 3 39 ['SnirBroshi', 'SuccessMoses', 'alreadydone', 'github-actions', 'grunweg', 'j-loreaux'] nobody
30-82373
30 days ago
36-43223
36 days ago
2-76065
2 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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra awaiting-author t-number-theory merge-conflict
label:t-algebra$
331/2 Mathlib/FieldTheory/RatFunc/AsPolynomial.lean,Mathlib/FieldTheory/RatFunc/Degree.lean,Mathlib/NumberTheory/RatFunc/Ostrowski.lean 3 32 ['MichaelStollBayreuth', 'alreadydone', 'github-actions', 'mariainesdff', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] MichaelStollBayreuth
assignee:MichaelStollBayreuth
30-79183
30 days ago
75-42424
75 days ago
2-38055
2 days
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-ring-theory awaiting-author merge-conflict 29/0 Mathlib/RingTheory/Spectrum/Prime/RingHom.lean 1 4 ['bwangpj', 'erdOne', 'github-actions', 'mathlib4-merge-conflict-bot'] nobody
30-68219
30 days ago
53-40760
53 days ago
0-4624
1 hour
32829 Hagb
author:Hagb
feat(Data/Finsupp/MonomialOrder): weaken `IsOrderedCancelAddMonoid` to `IsOrderedAddMonoid` `IsOrderedCancelAddMonoid syn` (`.iocam`) can be obtained from `IsOrderedAddMonoid syn` and other fields. --- - [ ] depends on: #32828 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR 11/2 Mathlib/Algebra/Order/Group/Defs.lean,Mathlib/Data/Finsupp/MonomialOrder.lean 2 5 ['Hagb', 'github-actions', 'mathlib4-dependent-issues-bot', 'vihdzp'] nobody
30-63702
30 days ago
unknown
unknown
32211 ADedecker
author:ADedecker
feat: inclusion from `ContDiffMapSupportedIn` to `TestFunction` is a topological embedding --- - [ ] depends on: #32210 - [x] depends on: #31806 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis blocked-by-other-PR merge-conflict 136/2 Mathlib/Analysis/Distribution/TestFunction.lean,Mathlib/Topology/UniformSpace/UniformEmbedding.lean 2 5 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
30-47313
30 days ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis large-import merge-conflict 191/0 Mathlib/Analysis/Distribution/ContDiffMapSupportedIn.lean,Mathlib/Analysis/Distribution/TestFunction.lean 2 3 ['github-actions', 'mathlib4-merge-conflict-bot'] nobody
30-47312
30 days ago
unknown
unknown
32602 adamtopaz
author:adamtopaz
feat: Refactor graph Work in progress --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP 1312/0 RefactorGraph/DAG.lean,RefactorGraph/Main.lean,RefactorGraph/Test.lean,lakefile.lean 4 1 ['github-actions'] nobody
30-41434
30 days ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) I found this being not-simp frustrating when talking about submodules over a valuation subring. merge-conflict t-algebra
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 26 ['artie2000', 'eric-wieser', 'github-actions', 'j-loreaux', 'kckennylau', 'leanprover-bot', 'leanprover-radar', 'linesthatinterlace', 'mathlib4-merge-conflict-bot', 'pechersky'] joelriou
assignee:joelriou
30-38311
30 days ago
51-74260
51 days ago
60-49993
60 days
32737 j-loreaux
author:j-loreaux
refactor: rename `MulAction` to `MonoidAction` Given that we now have [SemigroupAction](https://leanprover-community.github.io/mathlib4_docs/Mathlib/Algebra/Group/Action/Defs.html#SemigroupAction) we are in the unfortunate scenario that the name which seems to have less structure actually has *more* structure. This PR: 1. renames `MulAction` to `MonoidAction` to reflect this additional structure, as well as declarations referencing `MulAction` in their names. `Prop`-valued mixins in the `MulAction` namespace are also renamed (e.g., `MulAction.{IsMinimal,IsTopologicallyTransitive}` → `MonoidAction.{IsMinimal,IsTopologicallyTransitive`). 2. The additive version are also renamed (`AddAction` → `AddMonoidAction`) and the corresponding `Prop`-valued mixins. 3. does *not* rename modules with `MulAction` in the name 4. does *not* rename `DistribMulAction`, `SubMulAction`, `MulActionWithZero`, etc. If these need to happen, that can occur at a later time. 5. does *not* rename `SemigroupAction` to `MulAction`. Even if this rename is desired, because of the prevalence of `MulAction` in Mathlib, I think we should not conduct a move of this magnitude all at once. If we want to rename this to `MulAction`, we should wait for the 6 month embargo period during which time that name is deprecated, to give everyone downstream the opportunity to switch instead of silently breaking their builds. Of course, another potential name is `MulOneAction`, but I don't think that's too helpful. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict 3623/1862 Mathlib/Algebra/AddConstMap/Basic.lean,Mathlib/Algebra/AddTorsor/Basic.lean,Mathlib/Algebra/AddTorsor/Defs.lean,Mathlib/Algebra/Algebra/Equiv.lean,Mathlib/Algebra/Algebra/NonUnitalHom.lean,Mathlib/Algebra/Algebra/Subalgebra/Basic.lean,Mathlib/Algebra/Algebra/Subalgebra/Pointwise.lean,Mathlib/Algebra/Algebra/Tower.lean,Mathlib/Algebra/Algebra/Unitization.lean,Mathlib/Algebra/BigOperators/Group/Finset/Basic.lean,Mathlib/Algebra/BigOperators/Group/Finset/Defs.lean,Mathlib/Algebra/BigOperators/Group/Finset/Pi.lean,Mathlib/Algebra/BigOperators/Group/Finset/Preimage.lean,Mathlib/Algebra/BigOperators/GroupWithZero/Action.lean,Mathlib/Algebra/Category/ModuleCat/ChangeOfRings.lean,Mathlib/Algebra/Category/ModuleCat/FilteredColimits.lean,Mathlib/Algebra/Colimit/DirectLimit.lean,Mathlib/Algebra/Field/Action/ConjAct.lean,Mathlib/Algebra/Field/Subfield/Basic.lean,Mathlib/Algebra/FreeMonoid/Basic.lean,Mathlib/Algebra/GradedMonoid.lean,Mathlib/Algebra/GradedMulAction.lean,Mathlib/Algebra/Group/Action/Basic.lean,Mathlib/Algebra/Group/Action/Defs.lean,Mathlib/Algebra/Group/Action/End.lean,Mathlib/Algebra/Group/Action/Equidecomp.lean,Mathlib/Algebra/Group/Action/Faithful.lean,Mathlib/Algebra/Group/Action/Hom.lean,Mathlib/Algebra/Group/Action/Opposite.lean,Mathlib/Algebra/Group/Action/Option.lean,Mathlib/Algebra/Group/Action/Pi.lean,Mathlib/Algebra/Group/Action/Pointwise/Finset.lean,Mathlib/Algebra/Group/Action/Pointwise/Set/Basic.lean,Mathlib/Algebra/Group/Action/Pointwise/Set/Finite.lean,Mathlib/Algebra/Group/Action/Pretransitive.lean,Mathlib/Algebra/Group/Action/Prod.lean,Mathlib/Algebra/Group/Action/Sigma.lean,Mathlib/Algebra/Group/Action/Sum.lean,Mathlib/Algebra/Group/Action/TransferInstance.lean,Mathlib/Algebra/Group/Action/TypeTags.lean,Mathlib/Algebra/Group/Action/Units.lean,Mathlib/Algebra/Group/Conj.lean,Mathlib/Algebra/Group/End.lean,Mathlib/Algebra/Group/Equiv/Finite.lean,Mathlib/Algebra/Group/Nat/Range.lean,Mathlib/Algebra/Group/Pointwise/Finset/Basic.lean,Mathlib/Algebra/Group/Pointwise/Finset/Density.lean,Mathlib/Algebra/Group/Pointwise/Finset/Scalar.lean,Mathlib/Algebra/Group/Pointwise/Set/Basic.lean,Mathlib/Algebra/Group/Pointwise/Set/Card.lean,Mathlib/Algebra/Group/Pointwise/Set/Finite.lean,Mathlib/Algebra/Group/Pointwise/Set/Lattice.lean,Mathlib/Algebra/Group/Pointwise/Set/Scalar.lean,Mathlib/Algebra/Group/Shrink.lean,Mathlib/Algebra/Group/Subgroup/Actions.lean,Mathlib/Algebra/Group/Subgroup/Basic.lean,Mathlib/Algebra/Group/Subgroup/Pointwise.lean,Mathlib/Algebra/Group/Submonoid/Membership.lean,Mathlib/Algebra/Group/Submonoid/MulAction.lean,Mathlib/Algebra/Group/Submonoid/Pointwise.lean,Mathlib/Algebra/Group/TransferInstance.lean,Mathlib/Algebra/Group/TypeTags/Finite.lean,Mathlib/Algebra/GroupWithZero/Action/Basic.lean,Mathlib/Algebra/GroupWithZero/Action/ConjAct.lean,Mathlib/Algebra/GroupWithZero/Action/Defs.lean,Mathlib/Algebra/GroupWithZero/Action/End.lean,Mathlib/Algebra/GroupWithZero/Action/Faithful.lean,Mathlib/Algebra/GroupWithZero/Action/Opposite.lean,Mathlib/Algebra/GroupWithZero/Action/Pi.lean,Mathlib/Algebra/GroupWithZero/Action/Pointwise/Finset.lean,Mathlib/Algebra/GroupWithZero/Action/Pointwise/Set.lean,Mathlib/Algebra/GroupWithZero/Action/Prod.lean,Mathlib/Algebra/GroupWithZero/Action/TransferInstance.lean,Mathlib/Algebra/GroupWithZero/Action/Units.lean,Mathlib/Algebra/GroupWithZero/NonZeroDivisors.lean,Mathlib/Algebra/GroupWithZero/Pointwise/Finset.lean,Mathlib/Algebra/GroupWithZero/Pointwise/Set/Basic.lean,Mathlib/Algebra/GroupWithZero/Pointwise/Set/Card.lean,Mathlib/Algebra/GroupWithZero/Subgroup.lean,Mathlib/Algebra/GroupWithZero/Submonoid/Pointwise.lean,Mathlib/Algebra/GroupWithZero/TransferInstance.lean,Mathlib/Algebra/GroupWithZero/Units/Lemmas.lean,Mathlib/Algebra/Module/Congruence/Defs.lean,Mathlib/Algebra/Module/Defs.lean,Mathlib/Algebra/Module/Equiv/Basic.lean,Mathlib/Algebra/Module/GradedModule.lean,Mathlib/Algebra/Module/LinearMap/Defs.lean,Mathlib/Algebra/Module/LinearMap/End.lean,Mathlib/Algebra/Module/PUnit.lean,Mathlib/Algebra/Module/PointwisePi.lean,Mathlib/Algebra/Module/Rat.lean,Mathlib/Algebra/Module/RingHom.lean,Mathlib/Algebra/Module/Submodule/Basic.lean,Mathlib/Algebra/Module/Submodule/Defs.lean,Mathlib/Algebra/Module/Submodule/Invariant.lean,Mathlib/Algebra/Module/Submodule/LinearMap.lean,Mathlib/Algebra/Module/Submodule/Pointwise.lean,Mathlib/Algebra/Module/ULift.lean,Mathlib/Algebra/Order/Group/Action.lean,Mathlib/Algebra/Order/Group/Action/End.lean 349 3 ['github-actions', 'mathlib4-merge-conflict-bot'] nobody
29-86073
29 days ago
31-4588
31 days ago
2-47999
2 days
31926 kim-em
author:kim-em
experiment: use `grind` more in #31923 - [x] depends on #31929 4/4 Mathlib/Data/Finsupp/Basic.lean,Mathlib/Data/Finsupp/Sigma.lean,Mathlib/Data/Set/Sigma.lean,Mathlib/Logic/Embedding/Basic.lean 4 4 ['github-actions', 'mathlib4-merge-conflict-bot'] nobody
29-76688
29 days ago
29-76688
29 days ago
0-33519
9 hours
32942 kim-em
author:kim-em
feat(CategoryTheory/Monoidal/Rigid): tensor product of exact pairings This PR adds the tensor product construction for exact pairings in rigid monoidal categories: - `ExactPairing.tensor`: Given exact pairings `(X₁, Y₁)` and `(X₂, Y₂)`, we get an exact pairing `(X₁ ⊗ X₂, Y₂ ⊗ Y₁)`. Note the reversed order in the second factor - this is essential for the monoidal structure of dual functors. - `HasRightDual.tensor` and `HasLeftDual.tensor`: If `X` and `Y` have duals, so does `X ⊗ Y` - `rightDual_tensor` and `leftDual_tensor` simp lemmas **Status:** The triangle equation proofs (`coevaluation_evaluation'` and `evaluation_coevaluation'`) are currently `sorry` - working on completing them. 🤖 Prepared with Claude Code t-category-theory WIP 28/0 Mathlib/CategoryTheory/Monoidal/Rigid/Basic.lean 1 1 ['github-actions'] nobody
29-72643
29 days ago
unknown
unknown
26608 vihdzp
author:vihdzp
feat(SetTheory/Cardinal/Aleph): `o.card ≤ ℵ_ o` and variants --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-set-theory 24/0 Mathlib/SetTheory/Cardinal/Aleph.lean 1 4 ['artie2000', 'github-actions', 'kckennylau', 'leanprover-community-bot-assistant', 'vihdzp'] alreadydone
assignee:alreadydone
29-66800
29 days ago
29-74567
29 days ago
59-56107
59 days
24050 Paul-Lez
author:Paul-Lez
feat(Data/Finsupp/Pointwise): generalise pointwise scalar multiplication of finsupps As pointed out by @eric-wieser, this creates an instance diamond with `SMul (α → β) (α →₀ (α → β))` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-data 7/4 Mathlib/Data/Finsupp/Pointwise.lean 1 10 ['Paul-Lez', 'eric-wieser', 'github-actions', 'kckennylau', 'pechersky'] pechersky
assignee:pechersky
29-59920
29 days ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-analysis t-meta large-import 12024/2 Mathlib.lean,Mathlib/Data/Seq/Basic.lean,Mathlib/Data/Seq/Defs.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/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/Corecursion.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/Inv.lean,Mathlib/Tactic/ComputeAsymptotics/Multiseries/Operations/Log.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,MathlibTest/compute_asymptotics.lean 38 12 ['github-actions', 'grunweg', 'mathlib4-dependent-issues-bot', 'ocfnash', 'vasnesterov'] nobody
29-58211
29 days ago
unknown
unknown
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 --- - [x] 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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis awaiting-author 164/0 Mathlib/Analysis/Distribution/ContDiffMapSupportedIn.lean 1 16 ['ADedecker', 'github-actions', 'j-loreaux', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] j-loreaux, sgouezel, urkud
assignee:urkud assignee:j-loreaux assignee:sgouezel
29-47191
29 days ago
29-48042
29 days ago
4-19917
4 days
31386 harahu
author:harahu
doc: demote repeated H1 headers to H2 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 221/5 Mathlib/CategoryTheory/Bicategory/Functor/StrictPseudofunctor.lean,Mathlib/MeasureTheory/Function/ConditionalExpectation/PullOut.lean,Mathlib/Tactic/Common.lean,Mathlib/Tactic/Linter/EmptyLine.lean,scripts/demote_docstring_headers.py,scripts/find_docstring_headers.py 6 6 ['github-actions', 'mathlib4-merge-conflict-bot'] nobody
29-39568
29 days ago
unknown
unknown
32828 Hagb
author:Hagb
feat(Algebra/Order/Group/Defs): add `IsOrderedAddMonoid.toIsOrderedCancelAddMonoid'` It is similar to `IsOrderedAddMonoid.toIsOrderedCancelAddMonoid`, while with different hypotheses. The conclusion `IsOrderedCancelMonoid α` on `IsOrderedAddMonoid.toIsOrderedCancelAddMonoid` still holds when the hypothesis `CommGroup α` is weakened to `CancelCommMonoid α` while `PartialOrder α` is strengthened to `LinearOrder α`. --- [`IsOrderedAddMonoid.toIsOrderedCancelAddMonoid`](https://leanprover-community.github.io/mathlib4_docs/find/?pattern=IsOrderedAddMonoid.toIsOrderedCancelAddMonoid#doc) and `IsOrderedAddMonoid.toIsOrderedCancelAddMonoid'`: https://github.com/leanprover-community/mathlib4/blob/97f78b1a4311fed1844b94f1c069219a48a098e1/Mathlib/Algebra/Order/Group/Defs.lean#L52-L62 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
4/0 Mathlib/Algebra/Order/Group/Defs.lean 1 1 ['artie2000', 'github-actions'] eric-wieser
assignee:eric-wieser
29-31268
29 days ago
33-7652
33 days ago
0-9883
2 hours
32717 adomani
author:adomani
perf: small speed up of the flexible linter This just rearranges an array accumulation. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-linter merge-conflict 7/8 Mathlib/Tactic/Linter/FlexibleLinter.lean 1 4 ['adomani', 'github-actions', 'leanprover-radar', 'mathlib4-merge-conflict-bot'] nobody
29-18536
29 days ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra large-import
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
28-79436
28 days ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) file-removed blocked-by-other-PR t-category-theory merge-conflict 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 6 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
28-50448
28 days ago
60-70351
60 days ago
0-8463
2 hours
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. --- - [x] depends on: #29284 [Extra lemmas in CategoryTheory.Core] --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) file-removed t-category-theory awaiting-author merge-conflict 209/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 25 ['Jlh18', 'dagurtomas', 'github-actions', 'joelriou', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
28-50447
28 days ago
35-49074
35 days ago
2-52111
2 days
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 --- - [x] depends on: #31908 - [x] depends on: #31910 - [x] depends on: #31942 - [x] depends on: #31947 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-measure-probability 266/2 Mathlib.lean,Mathlib/MeasureTheory/Integral/Bochner/Set.lean,Mathlib/MeasureTheory/Measure/Dirac.lean,Mathlib/MeasureTheory/Measure/Restrict.lean,Mathlib/Probability/Distributions/Binomial.lean,Mathlib/Probability/Moments/Variance.lean 6 52 ['DavidLedvinka', 'RemyDegenne', 'YaelDillies', 'github-actions', 'kex-y', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'pfaffelh', 'themathqueen'] kex-y
assignee:kex-y
28-48216
28 days ago
128-8981
128 days ago
24-73279
24 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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory large-import merge-conflict 133/46 Mathlib/CategoryTheory/Bicategory/InducedBicategory.lean,Mathlib/CategoryTheory/Category/Grpd.lean,Mathlib/CategoryTheory/ConcreteCategory/Bundled.lean 3 6 ['Jlh18', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
28-46933
28 days ago
unknown
unknown
33015 thorimur
author:thorimur
share: stress test plugins via pluginizing Mathlib.Init This PR is only created for conveniently sharing this branch via `gh` for the purpose of experimenting with plugins. There's no plan to make Mathlib.Init a plugin any time soon. :) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict 999/1080 Mathlib.lean,Mathlib/Algebra/Expr.lean,Mathlib/Algebra/HierarchyDesign.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Note.lean,Mathlib/CategoryTheory/Category/Init.lean,Mathlib/CategoryTheory/ConcreteCategory/Bundled.lean,Mathlib/Combinatorics/Matroid/Init.lean,Mathlib/Combinatorics/SimpleGraph/Init.lean,Mathlib/Control/Combinators.lean,Mathlib/Control/ULift.lean,Mathlib/Data/Array/Defs.lean,Mathlib/Data/Array/Extract.lean,Mathlib/Data/Finset/Attr.lean,Mathlib/Data/Int/DivMod.lean,Mathlib/Data/Int/Notation.lean,Mathlib/Data/List/Monad.lean,Mathlib/Data/Nat/BinaryRec.lean,Mathlib/Data/Nat/Init.lean,Mathlib/Data/Nat/Notation.lean,Mathlib/Data/Nat/NthRoot/Defs.lean,Mathlib/Data/Set/Defs.lean,Mathlib/Data/String/Defs.lean,Mathlib/Data/Sym/Sym2/Init.lean,Mathlib/Data/UInt.lean,Mathlib/Deprecated/Aliases.lean,Mathlib/Deprecated/Sort.lean,Mathlib/Lean/ContextInfo.lean,Mathlib/Lean/CoreM.lean,Mathlib/Lean/Elab/InfoTree.lean,Mathlib/Lean/Elab/Tactic/Meta.lean,Mathlib/Lean/Elab/Term.lean,Mathlib/Lean/EnvExtension.lean,Mathlib/Lean/Environment.lean,Mathlib/Lean/Exception.lean,Mathlib/Lean/Expr/Basic.lean,Mathlib/Lean/Expr/Rat.lean,Mathlib/Lean/GoalsLocation.lean,Mathlib/Lean/Json.lean,Mathlib/Lean/LinterCopies.lean,Mathlib/Lean/LinterCopiesTest.lean,Mathlib/Lean/LocalContext.lean,Mathlib/Lean/Meta.lean,Mathlib/Lean/Meta/Basic.lean,Mathlib/Lean/Meta/DiscrTree.lean,Mathlib/Lean/Meta/KAbstractPositions.lean,Mathlib/Lean/Meta/RefinedDiscrTree/Basic.lean,Mathlib/Lean/Meta/Simp.lean,Mathlib/Lean/Meta/Tactic/Rewrite.lean,Mathlib/Lean/Name.lean,Mathlib/Lean/PrettyPrinter/Delaborator.lean,Mathlib/Lean/Thunk.lean,Mathlib/Logic/Basic.lean,Mathlib/Logic/OpClass.lean,Mathlib/Tactic.lean,Mathlib/Tactic/AdaptationNote.lean,Mathlib/Tactic/ApplyCongr.lean,Mathlib/Tactic/ApplyWith.lean,Mathlib/Tactic/ArithMult/Init.lean,Mathlib/Tactic/Attr/Register.lean,Mathlib/Tactic/Basic.lean,Mathlib/Tactic/Bound/Init.lean,Mathlib/Tactic/CC/Lemmas.lean,Mathlib/Tactic/Cases.lean,Mathlib/Tactic/CasesM.lean,Mathlib/Tactic/CategoryTheory/CategoryStar.lean,Mathlib/Tactic/CategoryTheory/Coherence/Datatypes.lean,Mathlib/Tactic/Change.lean,Mathlib/Tactic/Check.lean,Mathlib/Tactic/Clean.lean,Mathlib/Tactic/ClearExcept.lean,Mathlib/Tactic/ClearExclamation.lean,Mathlib/Tactic/Clear_.lean,Mathlib/Tactic/Coe.lean,Mathlib/Tactic/Common.lean,Mathlib/Tactic/Constructor.lean,Mathlib/Tactic/Continuity/Init.lean,Mathlib/Tactic/Conv.lean,Mathlib/Tactic/Core.lean,Mathlib/Tactic/DepRewrite.lean,Mathlib/Tactic/Eqns.lean,Mathlib/Tactic/ErwQuestion.lean,Mathlib/Tactic/Eval.lean,Mathlib/Tactic/ExistsI.lean,Mathlib/Tactic/Explode/Datatypes.lean,Mathlib/Tactic/ExtendDoc.lean,Mathlib/Tactic/FailIfNoProgress.lean,Mathlib/Tactic/FastInstance.lean,Mathlib/Tactic/FieldSimp/Attr.lean,Mathlib/Tactic/Find.lean,Mathlib/Tactic/FindSyntax.lean,Mathlib/Tactic/Finiteness/Attr.lean,Mathlib/Tactic/FunProp/Decl.lean,Mathlib/Tactic/FunProp/Mor.lean,Mathlib/Tactic/FunProp/ToBatteries.lean,Mathlib/Tactic/GCongr/ForwardAttr.lean,Mathlib/Tactic/Generalize.lean,Mathlib/Tactic/GuardGoalNums.lean,Mathlib/Tactic/GuardHypNums.lean,Mathlib/Tactic/Have.lean,Mathlib/Tactic/HaveI.lean 211 0 [] nobody
28-45301
28 days ago
unknown
unknown
32772 tb65536
author:tb65536
feat(Data/Set/Card): criterion for `s.ncard ≤ (f '' s).ncard + 1` This PR gives a criterion `s.ncard ≤ (f '' s).ncard + 1` (note that we always have the inequality `(f '' s).ncard ≤ s.ncard`). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data 31/0 Mathlib/Data/Set/Card.lean 1 1 ['github-actions'] pechersky
assignee:pechersky
28-31260
28 days ago
34-14215
34 days ago
34-14035
34 days
32555 ksenono
author:ksenono
feat(Combinatorics/SimpleGraph/Matching): maximum and maximal matchings for Konig's theorem --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics new-contributor 127/1 Mathlib/Combinatorics/SimpleGraph/DegreeSum.lean,Mathlib/Combinatorics/SimpleGraph/Matching.lean 2 8 ['SnirBroshi', 'github-actions', 'ksenono'] awainverse
assignee:awainverse
28-19910
28 days ago
28-18983
28 days ago
38-43127
38 days
32570 ksenono
author:ksenono
feat(Combinatorics/SimpleGraph): bipartite subgraphs and vertex-disjoint graphs for Konig's theorem --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics new-contributor 22/0 Mathlib/Combinatorics/SimpleGraph/Bipartite.lean,Mathlib/Combinatorics/SimpleGraph/Subgraph.lean 2 10 ['SnirBroshi', 'github-actions'] kmill
assignee:kmill
28-19450
28 days ago
28-18542
28 days ago
38-18442
38 days
33020 FormulaRabbit81
author:FormulaRabbit81
chore(Topology): Deprecate file --- - [ ] depends on: #30851 deprecation [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology large-import merge-conflict 82/49 Mathlib/Topology/Compactness/HilbertCubeEmbedding.lean,Mathlib/Topology/MetricSpace/HausdorffAlexandroff.lean,Mathlib/Topology/MetricSpace/PiNat.lean 3 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
28-18404
28 days ago
28-18405
28 days ago
0-13670
3 hours
21447 erdOne
author:erdOne
feat(AlgebraicGeometry): the split algebraic torus --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-algebraic-geometry 419/0 Mathlib.lean,Mathlib/AlgebraicGeometry/Torus.lean 2 6 ['erdOne', 'github-actions', 'jcommelin', 'joelriou', 'mathlib4-merge-conflict-bot'] nobody
28-4972
28 days ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-analysis 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 8 ['ADedecker', 'faenuccio', 'github-actions', 'grunweg', 'yhx-12243'] nobody
27-82328
27 days ago
unknown
unknown
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 merge-conflict 101/0 Mathlib/Analysis/Convex/Between.lean,Mathlib/LinearAlgebra/AffineSpace/FiniteDimensional.lean,Mathlib/LinearAlgebra/AffineSpace/Independent.lean 3 6 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'ocfnash', 'zcyemi'] nobody
27-78523
27 days ago
48-57007
48 days ago
7-39599
7 days
25963 artie2000
author:artie2000
refactor(Algebra): uniform API for substructures * Add class for `SetLike` instances whose map preserves meets - the intended interpretation is substructures whose closure properties are preserved under intersection * Abstract out the `CompleteLattice` instance and `closure` adjunction on such instances This change unifies a significant part of the API for algebraic substructures. --- - [ ] depends on #32984 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) Original PR: https://github.com/leanprover-community/mathlib4/pull/20836 merge-conflict WIP t-algebra
label:t-algebra$
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 3 ['artie2000', 'github-actions', 'leanprover-community-bot-assistant'] nobody
27-62873
27 days ago
unknown
unknown
32845 jonasvanderschaaf
author:jonasvanderschaaf
feat(CategoryTheory): `GrothendieckTopology.yoneda` preserves certain (co)limits We prove that if every `J`-sheaf preserves limits of shape `Kᵒᵖ`, then `J.yoneda` preserves colimits of shape `K`, and the dual statement. We specialize to the case of finite products, and deduce that the inclusion of light profinite sets in light condensed sets preserves finite coproducts From [LeanCondensed](https://github.com/dagurtomas/LeanCondensed) --- Co-authored-by: Dagur Asgeirsson [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor WIP 108/0 Mathlib.lean,Mathlib/CategoryTheory/Limits/Preserves/Shapes/Products.lean,Mathlib/CategoryTheory/Sites/PreservesLimits.lean,Mathlib/CategoryTheory/Sites/Subcanonical.lean,Mathlib/Condensed/Light/Functors.lean 5 1 ['github-actions'] nobody
27-61031
27 days ago
unknown
unknown
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) - [ ] depends on: #33061 **The next PR is here:** #31670 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology new-contributor awaiting-author blocked-by-other-PR 293/1 Mathlib.lean,Mathlib/Topology/Order/ScottTopology.lean,Mathlib/Topology/Order/ScottTopologyDCPO.lean,docs/references.bib 4 39 ['b-mehta', 'edwin1729', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'plp127'] b-mehta
assignee:b-mehta
27-43666
27 days ago
47-73851
47 days ago
5-43456
5 days
32679 YaelDillies
author:YaelDillies
chore(Data/Sym2): improve defeq of `diagSet` #30559 introduced a regression on the defeqs in the `SimpleGraph` API. This PR fixes it. From LeanCamCombi --- I personally think this new `diagSet` definition is unnecessary: `{e | e.IsDiag}` is not much longer to write than `Sym2.diagSet` and more transparent, but whatever. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data 52/41 Mathlib/Combinatorics/SimpleGraph/Basic.lean,Mathlib/Combinatorics/SimpleGraph/DeleteEdges.lean,Mathlib/Combinatorics/SimpleGraph/Operations.lean,Mathlib/Data/Sym/Card.lean,Mathlib/Data/Sym/Sym2.lean 5 9 ['SnirBroshi', 'YaelDillies', 'b-mehta', 'github-actions', 'mathlib4-merge-conflict-bot', 'vihdzp'] pechersky
assignee:pechersky
27-42874
27 days ago
27-41048
27 days ago
33-80987
33 days
32941 kim-em
author:kim-em
feat(GroupTheory/Artin): add Artin groups and braid groups This PR introduces Artin groups (also called Artin-Tits groups) as presented groups associated to Coxeter matrices, and defines braid groups as the special case of type A. ## Main definitions In `Mathlib/GroupTheory/Artin/Basic.lean`: - `CoxeterMatrix.ArtinGroup`: The Artin group associated to a Coxeter matrix - `CoxeterMatrix.artinGenerator`: The generators of the Artin group - `CoxeterMatrix.artinLift`: The universal property of Artin groups In `Mathlib/GroupTheory/Artin/Braid.lean`: - `CoxeterMatrix.typeA`: The Coxeter matrix of type A_n - `BraidGroup n`: The braid group B_n on n strands - `BraidGroup.σ`: The standard Artin generators - `BraidGroup.toPermHom`: The canonical surjection B_n → S_n - `BraidGroup.uniqueZero`, `uniqueOne`: B_0 and B_1 are trivial - `BraidGroup.equivIntTwo`: B_2 ≃* ℤ 🤖 Prepared with Claude Code t-group-theory 567/0 Mathlib.lean,Mathlib/Algebra/Group/End.lean,Mathlib/Algebra/Group/Subgroup/Basic.lean,Mathlib/GroupTheory/Artin/Basic.lean,Mathlib/GroupTheory/Artin/Braid.lean,Mathlib/GroupTheory/Coxeter/Matrix.lean,Mathlib/GroupTheory/Coxeter/Perm.lean,Mathlib/GroupTheory/FreeGroup/Basic.lean,Mathlib/GroupTheory/PresentedGroup.lean 9 11 ['github-actions', 'kim-em', 'robin-carlier', 'themathqueen'] nobody
27-16702
27 days ago
unknown
unknown
32938 0xTerencePrime
author:0xTerencePrime
feat(Order/LocallyFinite): prove DenselyOrdered and LocallyFiniteOrder are incompatible ## Summary This PR proves that a nontrivial densely ordered linear order cannot be locally finite. ## Main results * `not_locallyFiniteOrder`: A densely ordered locally finite linear order must be subsingleton. * `not_locallyFiniteOrder_of_nontrivial`: The main theorem - incompatibility of the two properties. Note: This implementation imports `Mathlib.Order.Interval.Set.Infinite` to reuse the existing `Set.Icc_infinite` theorem, ensuring standard library consistency. ## Mathematical content The key insight is that in a densely ordered type, we can always find a new element between any two distinct elements. This means any nontrivial interval contains infinitely many elements. However, `LocallyFiniteOrder` requires intervals to be finite. This contradiction implies that such a type cannot exist (unless it is trivial). ## Motivation This resolves a TODO mentioned in #7987 (Data/Finset/LocallyFinite entry). ## Verification - [x] `lake build Mathlib.Order.LocallyFinite.Basic` passes - [x] `lake exe runLinter Mathlib.Order.LocallyFinite.Basic` passes t-order new-contributor awaiting-author 28/0 Mathlib/Order/Interval/Finset/Basic.lean 1 10 ['0xTerencePrime', 'CoolRmal', 'github-actions', 'jcommelin', 'plp127'] nobody
27-2388
27 days ago
27-2428
27 days ago
2-83075
2 days
33077 YaelDillies
author:YaelDillies
feat(Data/Rel): balls Define `SetRel.ball` and use it in place of `UniformSpace.ball`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-data 38/3 Mathlib/Data/Rel.lean,Mathlib/Topology/UniformSpace/Defs.lean 2 1 ['github-actions'] nobody
26-80773
26 days ago
unknown
unknown
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]. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-ring-theory easy merge-conflict 3/2 Mathlib/RingTheory/Extension/Presentation/Core.lean,Mathlib/RingTheory/Ideal/Quotient/Operations.lean 2 7 ['erdOne', 'github-actions', 'j-loreaux', 'mathlib4-merge-conflict-bot'] nobody
26-70450
26 days ago
69-56151
69 days ago
2-6478
2 days
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebraic-topology blocked-by-other-PR new-contributor 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
26-62193
26 days ago
unknown
unknown
21495 alreadydone
author:alreadydone
experiment: reducible HasQuotient.quotient' --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP bench-after-CI merge-conflict 2/0 Mathlib/Algebra/Quotient.lean 1 2 ['github-actions', 'mathlib4-merge-conflict-bot'] nobody
26-55769
26 days ago
unknown
unknown
32532 SnirBroshi
author:SnirBroshi
feat(Combinatorics/SimpleGraph/Connectivity): connected components are maximally connected subsets/subgraphs --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics 32/0 Mathlib/Combinatorics/SimpleGraph/Connectivity/Connected.lean,Mathlib/Combinatorics/SimpleGraph/Connectivity/Subgraph.lean 2 2 ['github-actions', 'mathlib4-merge-conflict-bot'] awainverse
assignee:awainverse
26-39491
26 days ago
26-38660
26 days ago
39-5863
39 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`, a direct construction without ε-transitions. - Theorem `accepts_concat : (M1.concat M2).accepts = M1.accepts * M2.accepts`, showing the correctness of the construction. - Theorem `IsRegular.mul`, showing that regular languages are closed under concatenation. --- - [x] depends on: #31038 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-computability new-contributor maintainer-merge 104/7 Mathlib/Computability/NFA.lean 1 63 ['YaelDillies', 'ctchou', 'github-actions', 'lambda-fairy', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'rudynicolop'] YaelDillies
assignee:YaelDillies
26-39226
26 days ago
26-38270
26 days ago
45-11894
45 days
32698 farruhx
author:farruhx
feat(List): add aesop / simp annotations to selected lemmas for improved automation This PR adds `@[aesop safe]` and `@[simp]` annotations to a set of List lemmas whose proofs are routine and benefit from standardized automation. No statements or definitions are changed; only proof annotations are added. The lemmas updated in this PR are: * `or_exists_of_exists_mem_cons` * `append_subset_of_subset_of_subset` * `map_subset_iff` * `append_eq_has_append` * `append_right_injective` * `append_left_injective` * `reverse_surjective` * `reverse_bijective` * `mem_getLast?_append_of_mem_getLast?` * `mem_dropLast_of_mem_of_ne_getLast` * `idxOf_eq_length_iff` * `idxOf_append_of_mem` * `length_eraseP_add_one` The goal is to make these commonly used lemmas easier for `aesop`-based automation to resolve, while avoiding any interference with simp-normal-form lemmas or canonical rewrite rules. There are no API changes and no new theorems—only improved automation behavior. t-data new-contributor awaiting-author 18/1 Mathlib/Data/List/Basic.lean 1 8 ['artie2000', 'euprunin', 'farruhx', 'github-actions'] pechersky
assignee:pechersky
26-37157
26 days ago
26-37157
26 days ago
7-30937
7 days
32872 JovanGerb
author:JovanGerb
feat(Data/Real/Basic): don't expose the definition of `Real` This PR refactors the definition of `Real` using the module system, so that `Real` cannot be seen as a structure anymore. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data 141/250 Archive/Imo/Imo2013Q5.lean,Archive/Wiedijk100Theorems/BuffonsNeedle.lean,Counterexamples/SeminormLatticeNotDistrib.lean,Counterexamples/TopologistsSineCurve.lean,Mathlib/Analysis/SpecialFunctions/Gaussian/GaussianIntegral.lean,Mathlib/Data/Real/Basic.lean,MathlibTest/Complex.lean,MathlibTest/Continuity.lean,MathlibTest/Quaternion.lean,MathlibTest/Real.lean 10 2 ['github-actions', 'mathlib4-merge-conflict-bot'] nobody
26-35088
26 days ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-euclidean-geometry 157/0 Mathlib/Geometry/Euclidean/Angle/Oriented/Affine.lean 1 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] JovanGerb
assignee:JovanGerb
26-31276
26 days ago
29-41290
29 days ago
29-43242
29 days
32826 felixpernegger
author:felixpernegger
feat(Data/Tuple/Sort): Permutation is monotone iff its the identity Sort of permutation is its inverse + Permutation is monotone iff its the identity t-data new-contributor 19/0 Mathlib/Data/Fin/Tuple/Sort.lean 1 1 ['github-actions'] TwoFX
assignee:TwoFX
26-31272
26 days ago
30-75519
30 days ago
33-21577
33 days
29953 slashbade
author:slashbade
feat: add reap for experiment --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
26-19244
26 days ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) brownian t-measure-probability large-import 111/4 Mathlib/Data/Setoid/Partition.lean,Mathlib/MeasureTheory/Function/SimpleFunc.lean,Mathlib/MeasureTheory/Function/StronglyMeasurable/Basic.lean,Mathlib/MeasureTheory/MeasurableSpace/Basic.lean 4 21 ['CoolRmal', 'EtienneC30', 'github-actions', 'hanwenzhu', 'mathlib4-merge-conflict-bot'] EtienneC30
assignee:EtienneC30
25-83407
25 days ago
25-81917
25 days ago
47-53628
47 days
27817 zhuyizheng
author:zhuyizheng
feat: add IMO2025P1 Add a solution to IMO2025P1, the original problem statement from https://github.com/jsm28/IMOLean --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) IMO awaiting-author new-contributor merge-conflict 1310/0 Archive.lean,Archive/Imo/Imo2025Q1.lean 2 9 ['github-actions', 'kim-em', 'mathlib4-merge-conflict-bot', 'zhuyizheng'] dwrensha
assignee:dwrensha
25-69354
25 days ago
85-33922
85 days ago
54-69322
54 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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP awaiting-CI t-measure-probability file-removed FLT 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 23 ['YaelDillies', 'github-actions', 'kbuzzard', 'leanprover-community-bot-assistant', 'mathlib4-merge-conflict-bot', 'sgouezel'] nobody
25-44963
25 days ago
unknown
unknown
32739 Rida-Hamadani
author:Rida-Hamadani
chore(SimpleGraph): golf and improve style of `Subwalks.lean` maintaining the sub-walks file after the walk split, golfing some proofs --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics 11/18 Mathlib/Combinatorics/SimpleGraph/Walks/Subwalks.lean 1 1 ['github-actions', 'vlad902'] awainverse
assignee:awainverse
25-31245
25 days ago
34-180
34 days ago
34-0
34 days
32910 felixpernegger
author:felixpernegger
feat(Data/Nat/Choose): two binomial coefficient sum identities This PR proves two well-known sum identities around binomial coefficients. While there are probably hundreds of such identities, these two seem to be well known enough to be in mathlib (i.e. are mentioned in the Wikipedia [article](https://en.wikipedia.org/wiki/Binomial_coefficient#math_8) about binomial coefficients). new-contributor t-data 31/0 Mathlib/Data/Nat/Choose/Sum.lean,Mathlib/Data/Nat/Choose/Vandermonde.lean 2 1 ['github-actions'] TwoFX
assignee:TwoFX
25-31242
25 days ago
30-65061
30 days ago
30-64881
30 days
32989 kim-em
author:kim-em
fix(Tactic/Simps): skip @[defeq] inference for non-exposed definitions This PR makes `@[simps]` check whether the source definition's body is exposed before calling `inferDefEqAttr`. When the body is not exposed, we skip the `@[defeq]` inference to avoid validation errors. Without this fix, using `@[simps]` on a definition that is not `@[expose]`d produces an error like: ``` Theorem Foo_bar has a `rfl`-proof and was thus inferred to be `@[defeq]`, but validating that attribute failed: Not a definitional equality: the left-hand side ... is not definitionally equal to the right-hand side ... Note: This theorem is exported from the current module. This requires that all definitions that need to be unfolded to prove this theorem must be exposed. ``` The fix checks `(← getEnv).setExporting true |>.find? cfg.srcDeclName |>.any (·.hasValue)` to determine if the definition body is visible in the public scope, and only calls `inferDefEqAttr` if it is. 🤖 Prepared with Claude Code t-meta 40/2 Mathlib/Tactic/Simps/Basic.lean,MathlibTest/SimpsModule.lean 2 8 ['JovanGerb', 'github-actions', 'kim-em'] eric-wieser
assignee:eric-wieser
25-31241
25 days ago
26-32061
26 days ago
28-81065
28 days
33016 xgenereux
author:xgenereux
feat: RingHom.adjoinAlgebraMap Consider a tower of rings `A / B / C` and `b : B`, then there is a natural map from `A[b]` to `A[algebraMap B C b]` (adjoin `b` viewed as an element of `C`). This PR adds 3 versions, depending on whether we use `Algebra.adjoin` or `IntermediateField.adjoin`: - `Algebra.RingHom.adjoinAlgebraMap : Algebra.adjoin A {b} →+* Algebra.adjoin A {(algebraMap B C) b}` - `IntermediateField.RingHom.adjoinAlgebraMapOfAlgebra : Algebra.adjoin A {b} →+* A⟮((algebraMap B C) b)⟯` - `IntermediateField.RingHom.adjoinAlgebraMap : A⟮b⟯ →+* A⟮((algebraMap B C) b)⟯` Note: We create a new file for `Algebra.RingHom.adjoinAlgebraMap`, which is intended for results about adjoining singletons, because it is convenient to import `Algebra.Adjoin.Polynomial`. Co-authored-by: María Inés de Frutos Fernández <[mariaines.dff@gmail.com](mailto:mariaines.dff@gmail.com)> --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 103/0 Mathlib.lean,Mathlib/FieldTheory/IntermediateField/Adjoin/Algebra.lean,Mathlib/FieldTheory/IntermediateField/Adjoin/Defs.lean,Mathlib/RingTheory/Adjoin/Singleton.lean 4 1 ['github-actions'] bryangingechen
assignee:bryangingechen
25-31238
25 days ago
28-37014
28 days ago
28-36834
28 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 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] --> [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author new-contributor large-import 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
25-29725
25 days ago
115-84846
115 days ago
2-2914
2 days
30898 vihdzp
author:vihdzp
feat: characterization of `List.splitBy` --- - [x] depends on: #30892 Moved from #16837. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data 110/10 Mathlib/Data/List/Flatten.lean,Mathlib/Data/List/SplitBy.lean 2 6 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'vihdzp'] TwoFX
assignee:TwoFX
25-25272
25 days ago
25-22235
25 days ago
34-53081
34 days
33157 wwylele
author:wwylele
feat(Combinatorics): partitions and pentagonal numbers --- - [ ] depends on: #33143 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR 506/1 Mathlib.lean,Mathlib/Algebra/BigOperators/Ring/Finset.lean,Mathlib/Combinatorics/Enumerative/Partition/Basic.lean,Mathlib/Combinatorics/Enumerative/Partition/Pentagonal.lean,Mathlib/RingTheory/PowerSeries/Pentagonal.lean,Mathlib/Topology/Algebra/InfiniteSum/Pentagonal.lean,Mathlib/Topology/Algebra/InfiniteSum/Ring.lean,docs/1000.yaml 8 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
24-68844
24 days ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) please-adopt t-algebra large-import merge-conflict
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', 'mathlib4-dependent-issues-bot', 'mattrobball', 'pink10000', 'smorel394'] eric-wieser
assignee:eric-wieser
24-60443
24 days ago
unknown
unknown
32983 JovanGerb
author:JovanGerb
feat: use `LE.le` for subset relation in `Set`, `Finset`, `PSet`, `ZFSet` This PR allows the use of `⊆` notation while the underlying constant is `≤`. Similarly for `⊂`/`<`, `⊇`/`≥` and `⊃`/`>`. Hmm, seemingly still a lot of build failures --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict 248/159 Mathlib/Algebra/Group/Pointwise/Set/Basic.lean,Mathlib/Algebra/MonoidAlgebra/Support.lean,Mathlib/Combinatorics/Matroid/Basic.lean,Mathlib/Combinatorics/SetFamily/AhlswedeZhang.lean,Mathlib/Data/Finset/Defs.lean,Mathlib/Data/Finset/Filter.lean,Mathlib/Data/Finset/Image.lean,Mathlib/Data/Finset/Lattice/Basic.lean,Mathlib/Data/Fintype/Card.lean,Mathlib/Data/Multiset/ZeroCons.lean,Mathlib/Data/Rat/Star.lean,Mathlib/Data/Set/Basic.lean,Mathlib/Data/Set/Defs.lean,Mathlib/Data/Set/FiniteExhaustion.lean,Mathlib/Data/Set/Sups.lean,Mathlib/Data/SetLike/Basic.lean,Mathlib/Data/SetNotation.lean,Mathlib/MeasureTheory/SetSemiring.lean,Mathlib/Order/Birkhoff.lean,Mathlib/Order/BooleanAlgebra/Basic.lean,Mathlib/Order/Booleanisation.lean,Mathlib/Order/Bounds/Basic.lean,Mathlib/Order/CountableDenseLinearOrder.lean,Mathlib/Order/Filter/Basic.lean,Mathlib/Order/Heyting/Basic.lean,Mathlib/Order/RelClasses.lean,Mathlib/Order/SupIndep.lean,Mathlib/RingTheory/WittVector/StructurePolynomial.lean,Mathlib/SetTheory/ZFC/Basic.lean,Mathlib/SetTheory/ZFC/Class.lean,Mathlib/SetTheory/ZFC/PSet.lean,Mathlib/Topology/Compactness/SigmaCompact.lean,Mathlib/Topology/UniformSpace/Basic.lean 33 2 ['github-actions', 'mathlib4-merge-conflict-bot'] nobody
24-58455
24 days ago
unknown
unknown
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). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology new-contributor awaiting-author 110/18 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
24-15580
24 days ago
47-62982
47 days ago
8-9680
8 days
26923 oliver-butterley
author:oliver-butterley
feat(Dynamics/BirkhoffSum): add the pointwise ergodic theorem (Birkhoff's) The Pointwise Ergodic Theorem, also known as Birkhoff's Ergodic Theorem. Co-authored-by: Lua Viana Reis - [x] depends on: #26074 - [x] depends on: #26807 - [x] depends on: #26810 - [x] depends on: #26840 - [x] depends on: #26842 - [x] depends on: #26848 - [x] depends on: #26851 - [x] depends on: #26852 - [x] depends on: #26853 - [x] depends on: #27008 - [x] depends on: #28901 Zulip: [PR thread](https://leanprover.zulipchat.com/#narrow/channel/144837-PR-reviews/topic/.2326923.20The.20pointwise.20ergodic.20theorem.20.28Birkhoff's.29/with/527835158) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-dynamics new-contributor awaiting-author 398/0 Mathlib.lean,Mathlib/Dynamics/BirkhoffSum/Pointwise.lean 2 31 ['D-Thomine', 'github-actions', 'leanprover-community-bot-assistant', 'lua-vr', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'sgouezel', 'urkud'] sgouezel
assignee:sgouezel
24-5377
24 days ago
29-49695
29 days ago
98-42878
98 days
26484 peabrainiac
author:peabrainiac
feat(Geometry/Diffeology): basics of diffeological spaces Introduces diffeological spaces, smooth maps between them, the D-topology and the standard diffeology on finite-dimensional normed spaces. --- This PR continues the work from #21969. t-differential-geometry 491/0 Mathlib.lean,Mathlib/Geometry/Diffeology/Basic.lean,docs/references.bib 3 12 ['JovanGerb', 'github-actions', 'grunweg', 'lecopivo', 'mathlib4-merge-conflict-bot', 'peabrainiac'] ocfnash
assignee:ocfnash
24-462
24 days ago
25-34233
25 days ago
163-58726
163 days
26743 grunweg
author:grunweg
feat: product rule for Lie bracket on manifolds On the path towards geodesics and the Levi-Civita connection. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-differential-geometry 178/27 Mathlib/Geometry/Manifold/VectorField/LieBracket.lean,Mathlib/Geometry/Manifold/VectorField/Pullback.lean 2 4 ['github-actions', 'grunweg', 'mathlib4-merge-conflict-bot'] nobody
23-73681
23 days ago
unknown
unknown
33110 dagurtomas
author:dagurtomas
feat(CategoryTheory): adjoint functor theorems for presentable categories --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-category-theory 59/0 Mathlib/CategoryTheory/Presentable/AdjointFunctorTheorems.lean 1 2 ['github-actions', 'joelriou'] nobody
23-63332
23 days ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-euclidean-geometry 75/0 Mathlib/Geometry/Euclidean/Altitude.lean 1 4 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] JovanGerb
assignee:JovanGerb
23-31264
23 days ago
26-56741
26 days ago
26-56561
26 days
33031 chiyunhsu
author:chiyunhsu
feat(Combinatorics/Enumerative/Partition): add combinatorial proof of Euler's partition theorem The new file EulerComb.lean contains the combinatorial proof of Euler's partition theorem. The analytic proof of the theorem and its generalization of Glaisher's Theorem has already been formalized in [Glaisher.lean](https://github.com/leanprover-community/mathlib4/blob/master/Mathlib/Combinatorics/Enumerative/Partition/Glaisher.lean). The generalization of the combinatorial proof from this file to Glaisher's Theorem is within reach. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics new-contributor 531/0 Mathlib.lean,Mathlib/Combinatorics/Enumerative/Partition/EulerComb.lean 2 5 ['chiyunhsu', 'github-actions', 'tb65536', 'vihdzp'] b-mehta
assignee:b-mehta
23-31261
23 days ago
28-3017
28 days ago
28-2837
28 days
33082 AntoineChambert-Loir
author:AntoineChambert-Loir
feat(GroupTheory/SpecificGroups/Alternating/Simple): the alternating group on at least 5 letters is simple. This is the conclusion of the story of the proof of simplicity of the alternating group using the Iwasawa criterion. * `Equiv.Perm.iwasawaStructure_two`: the natural `IwasawaStructure` of `Equiv.Perm α` acting on `Nat.Combination α 2` Its commutative subgroups consist of the permutations with support in a given element of `Nat.Combination α 2`. They are cyclic of order 2. * `alternatingGroup_of_le_of_normal`: If `α` has at least 5 elements, then a nontrivial normal subgroup of `Equiv.Perm α` contains the alternating group. * `alternatingGroup.iwasawaStructure_three`: the natural `IwasawaStructure` of `alternatingGroup α` acting on `Nat.Combination α 3` Its commutative subgroups consist of the permutations with support in a given element of `Nat.Combination α 2`. They are cyclic of order 3. * `alternatingGroup.iwasawaStructure_three`: the natural `IwasawaStructure` of `alternatingGroup α` acting on `Nat.Combination α 4` Its commutative subgroups consist of the permutations of cycleType (2, 2) with support in a given element of `Nat.Combination α 2`. They have order 4 and exponent 2 (`IsKleinFour`). * `alternatingGroup.normal_subgroup_eq_bot_or_eq_top`: If `α` has at least 5 elements, then a nontrivial normal subgroup of `alternatingGroup` is `⊤`. * `alternatingGroup.isSimpleGroup`: If `α` has at least 5 elements, then `alternatingGroup α` is a simple group. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-group-theory large-import 821/13 Mathlib.lean,Mathlib/GroupTheory/GroupAction/SubMulAction/Combination.lean,Mathlib/GroupTheory/Perm/Cycle/Type.lean,Mathlib/GroupTheory/Perm/Support.lean,Mathlib/GroupTheory/SpecificGroups/Alternating.lean,Mathlib/GroupTheory/SpecificGroups/Alternating/Simple.lean,Mathlib/GroupTheory/SpecificGroups/KleinFour.lean 7 1 ['github-actions'] mattrobball
assignee:mattrobball
23-31256
23 days ago
26-59668
26 days ago
26-59488
26 days
33109 felixpernegger
author:felixpernegger
feat(Data/Nat/Choose): Binomial inversion This PR adds binomial inversion (also called binomial transform), which is a useful method for proving binomial identities. It is tricky to find direct references to binomial inversion, but for example [this](https://en.wikipedia.org/wiki/Binomial_transform#Binomial_convolution) Wikipedia article mentions it ("The formula"). The first theorem ```alternating_sum_choose_mul_of_alternating_sum_choose_mul``` could be refined (we only need the hypothesis ```h``` up to some point), but this seems to needlessly complicate it. new-contributor 107/0 Mathlib.lean,Mathlib/Data/Nat/Choose/Inversion.lean 2 4 ['felixpernegger', 'github-actions', 'wwylele'] dagurtomas
assignee:dagurtomas
23-31251
23 days ago
25-62272
25 days ago
26-4033
26 days
32497 themathqueen
author:themathqueen
chore: make `FiniteDimensional.complete 𝕜` an instance when `𝕜` is `RCLike` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis awaiting-bench 3/26 Mathlib/Analysis/InnerProductSpace/Adjoint.lean,Mathlib/Analysis/InnerProductSpace/Positive.lean 2 3 ['github-actions', 'leanprover-radar', 'themathqueen'] nobody
23-27354
23 days ago
unknown
unknown
33108 alreadydone
author:alreadydone
feat(Topology): `π₁(E⧸G)⧸π₁(E) ≃* G` for `E` path connected TODO: + finish last step (currently only `π₁(E⧸G) →* G` has been constructed) + characterization of the homomorphism + change of basepoint `e : E` leads to conjugation by `G` + if `G` is abelian then independent of choice of basepoint (and we can remove the ᵐᵒᵖ) + $\pi_1(S^1)\cong\mathbb{Z}$ + define winding number --- - [ ] depends on: #7596 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebraic-topology WIP t-topology merge-conflict 634/45 Mathlib.lean,Mathlib/Algebra/Group/Action/Pointwise/Set/Basic.lean,Mathlib/Algebra/Group/Submonoid/MulAction.lean,Mathlib/AlgebraicTopology/FundamentalGroupoid/Basic.lean,Mathlib/AlgebraicTopology/FundamentalGroupoid/FundamentalGroup.lean,Mathlib/Analysis/SpecialFunctions/Complex/Circle.lean,Mathlib/GroupTheory/GroupAction/SubMulAction.lean,Mathlib/Tactic/Translate/ToAdditive.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/Quotient.lean,Mathlib/Topology/Homotopy/Lifting.lean,Mathlib/Topology/Homotopy/Path.lean,Mathlib/Topology/Instances/AddCircle/Defs.lean 16 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
23-16627
23 days ago
unknown
unknown
33218 Blackfeather007
author:Blackfeather007
feat(Algebra): Define the associated graded ring to filtered ring Define the associated graded ring to a filtered ring. --- - [ ] depends on: #33217 migrated from https://github.com/leanprover-community/mathlib4/pull/26858 t-ring-theory new-contributor blocked-by-other-PR 450/0 Mathlib.lean,Mathlib/RingTheory/FilteredAlgebra/AssociatedGraded.lean 2 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
23-15619
23 days ago
unknown
unknown
33219 Blackfeather007
author:Blackfeather007
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: #33218 migrated from #26859 t-ring-theory new-contributor blocked-by-other-PR 563/0 Mathlib.lean,Mathlib/RingTheory/FilteredAlgebra/AssociatedGraded.lean 2 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
23-15511
23 days ago
unknown
unknown
33220 Blackfeather007
author:Blackfeather007
feat(Algebra): Define associated graded module Define the associated graded module to a filtered module. --- - [ ] depends on: #33218 migrated from #26860 t-ring-theory new-contributor blocked-by-other-PR 669/0 Mathlib.lean,Mathlib/RingTheory/FilteredAlgebra/AssociatedGraded.lean 2 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
23-15427
23 days ago
unknown
unknown
33227 Blackfeather007
author:Blackfeather007
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 [suzuka@misaka-yu.com](mailto:suzuka@misaka-yu.com) Co-authored-by: Yi Yuan @yuanyi-350 [kysyy1@126.com](mailto:kysyy1@126.com) Co-authored-by: Weichen Jiao @AlbertJ-314 [albertjiao314@gmail.com](mailto:albertjiao314@gmail.com) --- - [ ] depends on: #33226 migrated from #26869 t-ring-theory new-contributor blocked-by-other-PR 728/0 Mathlib.lean,Mathlib/RingTheory/FilteredAlgebra/AssociatedGraded.lean,Mathlib/RingTheory/FilteredAlgebra/Exactness.lean,Mathlib/RingTheory/FilteredAlgebra/FilteredHom.lean 4 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
23-13099
23 days ago
23-13100
23 days ago
0-206
3 minutes
33226 Blackfeather007
author:Blackfeather007
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 [suzuka@misaka-yu.com](mailto:suzuka@misaka-yu.com) Co-authored-by: Yi Yuan @yuanyi-350 [kysyy1@126.com](mailto:kysyy1@126.com) Co-authored-by: Weichen Jiao @AlbertJ-314 [albertjiao314@gmail.com](mailto:albertjiao314@gmail.com) --- - [ ] depends on: #33222 migrated from #26868 t-ring-theory new-contributor blocked-by-other-PR 529/0 Mathlib.lean,Mathlib/RingTheory/FilteredAlgebra/AssociatedGraded.lean,Mathlib/RingTheory/FilteredAlgebra/Exactness.lean,Mathlib/RingTheory/FilteredAlgebra/FilteredHom.lean 4 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
23-13097
23 days ago
23-13098
23 days ago
0-415
6 minutes
33225 Blackfeather007
author:Blackfeather007
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: #33220 - [ ] depends on: #33223 migrated from #26867 t-ring-theory new-contributor blocked-by-other-PR 1205/0 Mathlib.lean,Mathlib/RingTheory/FilteredAlgebra/AssociatedGraded.lean,Mathlib/RingTheory/FilteredAlgebra/FilteredHom.lean 3 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
23-13096
23 days ago
unknown
unknown
33224 Blackfeather007
author:Blackfeather007
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: #33219 - [ ] depends on: #33223 migrated from #26863 t-ring-theory new-contributor blocked-by-other-PR 1055/0 Mathlib.lean,Mathlib/RingTheory/FilteredAlgebra/AssociatedGraded.lean,Mathlib/RingTheory/FilteredAlgebra/FilteredHom.lean 3 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
23-13094
23 days ago
23-13095
23 days ago
0-978
16 minutes
33223 Blackfeather007
author:Blackfeather007
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 [suzuka@misaka-yu.com](mailto:suzuka@misaka-yu.com) Co-authored-by: Yi Yuan @yuanyi-350 [kysyy1@126.com](mailto:kysyy1@126.com) Co-authored-by: Weichen Jiao @AlbertJ-314 [albertjiao314@gmail.com](mailto:albertjiao314@gmail.com) --- - [ ] depends on: #33218 - [ ] depends on: #33222 migrated from #26862 t-ring-theory new-contributor blocked-by-other-PR 824/0 Mathlib.lean,Mathlib/RingTheory/FilteredAlgebra/AssociatedGraded.lean,Mathlib/RingTheory/FilteredAlgebra/FilteredHom.lean 3 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
23-13091
23 days ago
23-13094
23 days ago
0-1162
19 minutes
33222 Blackfeather007
author:Blackfeather007
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 [suzuka@misaka-yu.com](mailto:suzuka@misaka-yu.com) Co-authored-by: Yi Yuan @yuanyi-350 [kysyy1@126.com](mailto:kysyy1@126.com) Co-authored-by: Weichen Jiao @AlbertJ-314 [albertjiao314@gmail.com](mailto:albertjiao314@gmail.com) --- - [ ] depends on: #33217 migrated from #26861 new-contributor t-ring-theory blocked-by-other-PR 368/0 Mathlib.lean,Mathlib/RingTheory/FilteredAlgebra/AssociatedGraded.lean,Mathlib/RingTheory/FilteredAlgebra/FilteredHom.lean 3 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
23-13090
23 days ago
23-13091
23 days ago
0-1375
22 minutes
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis delegated 191/0 Mathlib.lean,Mathlib/Analysis/InnerProductSpace/Adjoint.lean,Mathlib/Analysis/InnerProductSpace/Coalgebra.lean,Mathlib/Analysis/InnerProductSpace/TensorProduct.lean,Mathlib/LinearAlgebra/TensorProduct/Associator.lean 5 47 ['github-actions', 'j-loreaux', 'mathlib-bors', 'mathlib4-merge-conflict-bot', 'ocfnash', 'themathqueen'] ocfnash
assignee:ocfnash
22-57808
22 days ago
36-54752
36 days ago
41-28400
41 days
33134 faenuccio
author:faenuccio
feat(Normed/Module/WeakDual): add Goldstine lemma We add Goldstine lemma stating that the weak*-closure of the image in the double dual of the unit ball coincides with the unit ball. As a corollary we derive that the image of `inclusionInDoubleDual` is weak*-dense. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-analysis 148/3 Mathlib/Analysis/Normed/Module/WeakDual.lean,Mathlib/Topology/Algebra/Module/WeakDual.lean,docs/references.bib 3 2 ['github-actions'] nobody
22-53878
22 days ago
unknown
unknown
33178 gw90
author:gw90
feat(Analysis/CStarAlgebra/Spectrum): Adding lemmas that the CStarAlgebra norm equals the square root of the spectral radius of star a * a Adds lemmas that the ||a||^2_A=sqrt(spectralRadius C (star a * a)). I think it would be helpful to have these lemmas available in Mathlib. It'll help with some of the other things I'm working on. Feel free to move them to a different file or rename them as you see fit. new-contributor t-analysis awaiting-author 24/0 Mathlib/Analysis/CStarAlgebra/Spectrum.lean 1 15 ['github-actions', 'gw90', 'themathqueen', 'vihdzp'] nobody
22-51358
22 days ago
24-26977
24 days ago
0-14336
3 hours
33126 CoolRmal
author:CoolRmal
feat: function composition preserves boundedness This PR adds the following theorem: if the range of a function `g` is bounded above, then `g ∘ f` is bounded above for all functions `f`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order 12/0 Mathlib/Order/Bounds/Basic.lean 1 1 ['github-actions'] bryangingechen
assignee:bryangingechen
22-31252
22 days ago
25-71900
25 days ago
25-71720
25 days
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 - [ ] depends on: #33249 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP blocked-by-other-PR t-combinatorics 825/0 Mathlib.lean,Mathlib/Combinatorics/SimpleGraph/GirthDiam.lean 2 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
22-25409
22 days ago
unknown
unknown
28462 joelriou
author:joelriou
feat(AlgebraicTopology/SimplicialSet): the relative cell complex attached to a rank function for a pairing WIP From https://github.com/joelriou/topcat-model-category --- - [x] depends on: #32515 - [x] depends on: #32517 - [x] depends on: #32178 - [x] depends on: #32180 - [x] depends on: #31122 - [x] depends on: #28351 - [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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebraic-topology WIP 410/0 Mathlib.lean,Mathlib/AlgebraicTopology/SimplicialSet/AnodyneExtensions/IsUniquelyCodimOneFace.lean,Mathlib/AlgebraicTopology/SimplicialSet/AnodyneExtensions/RelativeCellComplex.lean,Mathlib/AlgebraicTopology/SimplicialSet/Boundary.lean,Mathlib/AlgebraicTopology/SimplicialSet/Horn.lean,Mathlib/AlgebraicTopology/SimplicialSet/Simplices.lean,Mathlib/AlgebraicTopology/SimplicialSet/StdSimplex.lean,Mathlib/AlgebraicTopology/SimplicialSet/Subcomplex.lean,Mathlib/AlgebraicTopology/SimplicialSet/SubcomplexEvaluation.lean,Mathlib/Data/Fintype/Basic.lean,Mathlib/Order/Fin/Basic.lean 11 9 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
21-74173
21 days ago
unknown
unknown
33249 Rida-Hamadani
author:Rida-Hamadani
feat(SimpleGraph): `take` is path if original walk is path Proves that taking or dropping the first `n` consecution darts from a path gives another path. --- - [ ] depends on: #26614 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR t-combinatorics 76/0 Mathlib/Combinatorics/SimpleGraph/Paths.lean,Mathlib/Combinatorics/SimpleGraph/Walks/Operations.lean,Mathlib/Combinatorics/SimpleGraph/Walks/Subwalks.lean,Mathlib/Data/List/Infix.lean 4 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
21-59495
21 days ago
unknown
unknown
32160 SnirBroshi
author:SnirBroshi
feat(Combinatorics/SimpleGraph/Walks): helper theorems about `darts` and `support` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics 33/1 Mathlib/Combinatorics/SimpleGraph/Walks/Basic.lean,Mathlib/Combinatorics/SimpleGraph/Walks/Traversal.lean 2 1 ['github-actions'] kmill
assignee:kmill
21-46914
21 days ago
21-46054
21 days ago
49-22904
49 days
33147 SnirBroshi
author:SnirBroshi
feat(Combinatorics/SimpleGraph/Coloring): add a few missing instances (`IsEmpty`/`Nontrivial`/`Infinite`) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics 22/0 Mathlib/Combinatorics/SimpleGraph/Coloring.lean,Mathlib/Combinatorics/SimpleGraph/Maps.lean 2 1 ['github-actions'] b-mehta
assignee:b-mehta
21-31266
21 days ago
25-23536
25 days ago
25-23356
25 days
33269 urkud
author:urkud
feat(MeasureTheory/Covering): generalize some lemmas to outer measures --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-measure-probability 29/19 Mathlib/MeasureTheory/Covering/Differentiation.lean,Mathlib/MeasureTheory/Covering/VitaliFamily.lean 2 1 ['github-actions'] nobody
21-15002
21 days ago
unknown
unknown
31092 FlAmmmmING
author:FlAmmmmING
feat(Algebra/Group/ForwardDiff.lean): Add theorem `sum_shift_eq_fwdDiff_iter`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra new-contributor
label:t-algebra$
17/1 Mathlib/Algebra/Group/ForwardDiff.lean 1 18 ['BeibeiX0', 'FlAmmmmING', 'Ruben-VandeVelde', 'dagurtomas', 'github-actions', 'mathlib4-merge-conflict-bot'] dagurtomas
assignee:dagurtomas
21-6634
21 days ago
21-5473
21 days ago
46-81323
46 days
33121 SnirBroshi
author:SnirBroshi
feat(Combinatorics/SimpleGraph/Hasse): paths in a graph are isomorphic to path graphs --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics large-import 38/1 Mathlib/Combinatorics/SimpleGraph/Hasse.lean 1 1 ['github-actions'] b-mehta
assignee:b-mehta
20-79235
20 days ago
20-78270
20 days ago
25-84611
25 days
33138 gasparattila
author:gasparattila
chore(MeasureTheory/Measure/Stieltjes): remove `backward.privateInPublic` In #32482, some definitions in this file were rewritten using private declarations. However, this made `StieltjesFunction.length` unusable, since its API uses private declarations even in statements. This PR fixes this by problem by specializing `length_eq` to `NoMinOrder` and adding a new lemma for the `OrderBot` case. The other lemmas involving the private declarations are made private, except for `length_subadditive_Icc_Ioo`, which is reverted to the previous statement. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-measure-probability tech debt awaiting-author 35/30 Mathlib/MeasureTheory/Measure/Stieltjes.lean 1 6 ['github-actions', 'grunweg', 'sgouezel', 'vihdzp'] sgouezel
assignee:sgouezel
20-42331
20 days ago
20-42331
20 days ago
5-472
5 days
33211 Komyyy
author:Komyyy
doc(Order/Filter/*): outdated documents `f ×ˢ g` is not an notation of `Filter.prod` anymore, but [a notation class](https://leanprover-community.github.io/mathlib4_docs/Mathlib/Order/Filter/Defs.html#Filter.instSProd). Also, some definitions were moved to `Mathlib.Order.Filter.Defs`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) documentation t-order 6/10 Mathlib/Order/Filter/Curry.lean,Mathlib/Order/Filter/Pi.lean,Mathlib/Order/Filter/Prod.lean 3 6 ['Komyyy', 'github-actions', 'plp127'] bryangingechen
assignee:bryangingechen
20-31255
20 days ago
21-26899
21 days ago
23-30281
23 days
33043 euprunin
author:euprunin
chore: golf using `grind` and `simp` --- The goal of this golfing PR is to decrease the number of times lemmas are called explicitly (replacing calls to lemmas with calls to tactics). Any decrease in compilation time is a welcome side effect, although it is not a primary objective. Trace profiling results (shown if ≥10 ms before or after): * `CategoryTheory.MorphismProperty.isomorphisms_op`: <10 ms before, <10 ms after 🎉 * `Nat.ordProj_self_pow`: 23 ms before, <10 ms after 🎉 * `Pell.eq_pow_of_pell_lem`: 614 ms before, 658 ms after * `WittVector.RecursionBase.solution_spec'`: 60 ms before, 135 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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author 5/22 Mathlib/CategoryTheory/MorphismProperty/Basic.lean,Mathlib/Data/Nat/Factorization/Basic.lean,Mathlib/NumberTheory/PellMatiyasevic.lean,Mathlib/RingTheory/WittVector/FrobeniusFractionField.lean 4 2 ['github-actions', 'jcommelin'] nobody
20-16730
20 days ago
27-5857
27 days ago
0-59418
16 hours
32627 dagurtomas
author:dagurtomas
feat(Condensed): the functor from light profinite sets preserves effective epimorphisms From [LeanCondensed](https://github.com/dagurtomas/LeanCondensed) --- - [x] depends on: #32085 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-condensed 80/0 Mathlib.lean,Mathlib/Condensed/EffectiveEpi.lean,Mathlib/Condensed/Light/EffectiveEpi.lean 3 4 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'robin-carlier'] nobody
19-76322
19 days ago
19-76322
19 days ago
2-64010
2 days
33307 grunweg
author:grunweg
Orientable manifolds updated --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-differential-geometry 377/4 Mathlib.lean,Mathlib/Geometry/Manifold/Instances/Real.lean,Mathlib/Geometry/Manifold/Orientable.lean 3 2 ['github-actions'] nobody
19-73243
19 days ago
unknown
unknown
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 WIP blocked-by-other-PR t-order awaiting-CI merge-conflict 12/0 Mathlib/Algebra/Order/GroupWithZero/Unbundled/Basic.lean 1 48 ['Vierkantor', 'YaelDillies', 'faenuccio', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
19-72546
19 days ago
unknown
unknown
33313 SnirBroshi
author:SnirBroshi
feat(Combinatorics/SimpleGraph/EdgeColoring): create a basic edge-coloring API --- Future work (which I'm working on): - Relating degrees to edge-colorability (`G.maxDegree ≤ G.chromaticIndex`) - [Vizing's theorem](https://en.wikipedia.org/wiki/Vizing%27s_theorem) (`G.chromaticIndex ≤ G.maxDegree + 1`) - `chromaticIndex ⊤ = (if Even #V then #V - 1 else #V)` - [ ] depends on: #33292 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-combinatorics blocked-by-other-PR 307/4 Mathlib.lean,Mathlib/Combinatorics/SimpleGraph/EdgeColoring.lean,Mathlib/Combinatorics/SimpleGraph/LineGraph.lean,Mathlib/Data/Sym/Sym2.lean 4 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
19-61120
19 days ago
unknown
unknown
5934 eric-wieser
author:eric-wieser
feat: port Data.Rat.MetaDefs --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) This needs some eyes from people familiar with Qq merge-conflict help-wanted mathlib-port t-meta 183/0 Mathlib.lean,Mathlib/Data/Rat/MetaDefs.lean,test/rat.lean 3 5 ['eric-wieser', 'gebner', 'vihdzp'] nobody
19-53188
19 days ago
unknown
unknown
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` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-CI 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 1 ['vihdzp'] nobody
19-53085
19 days ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) please-adopt WIP t-algebra merge-conflict
label:t-algebra$
588/0 Mathlib.lean,Mathlib/LinearAlgebra/Matrix/SVD/Defs.lean,Mathlib/LinearAlgebra/Matrix/SVD/Reindex.lean 3 116 ['MohanadAhmed', 'Vierkantor', 'alexjbest', 'eric-wieser', 'j-loreaux', 'jcommelin', 'mathlib4-merge-conflict-bot', 'sgouezel', 'vihdzp'] nobody
19-52715
19 days ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-euclidean-geometry blocked-by-other-PR 200/0 Mathlib/Geometry/Euclidean/Altitude.lean,Mathlib/Geometry/Euclidean/Incenter.lean 2 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
19-49874
19 days ago
45-70775
45 days ago
0-1997
33 minutes
4127 kmill
author:kmill
refactor: create HasAdj class, define Digraph, and generalize some SimpleGraph API --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-combinatorics 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 2 ['SnirBroshi', 'vihdzp'] nobody
19-49060
19 days ago
unknown
unknown
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory new-contributor awaiting-author 527/0 Mathlib.lean,Mathlib/CategoryTheory/Bicategory/LaxSlice.lean 2 12 ['dagurtomas', 'github-actions', 'jjtowery', 'robin-carlier'] dagurtomas
assignee:dagurtomas
19-41576
19 days ago
unknown
unknown
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 awaiting-author t-order merge-conflict 14/0 Mathlib/Order/Directed.lean 1 5 ['github-actions', 'j-loreaux', 'mathlib4-merge-conflict-bot', 'plp127'] nobody
19-32793
19 days ago
unknown
unknown
33248 vihdzp
author:vihdzp
refactor(MeasureTheory/Measure/Stieltjes): simpler definition of `botSet` --- Arguably we could get rid of `botSet` altogether, but in either case this is still an improvement. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-measure-probability 13/19 Mathlib/MeasureTheory/Measure/Stieltjes.lean 1 1 ['github-actions'] EtienneC30
assignee:EtienneC30
19-31260
19 days ago
21-65987
21 days ago
21-65916
21 days
32546 anishrajeev
author:anishrajeev
feat(ModelTheory): Prove compactness of the type space Define the space of types and prove various topological properties of it (zero dimensional, totally separated, compact, baire). The goal is to formalize the proof of the Omitting Types Theorem - [ ] depends on: #32215 t-logic new-contributor blocked-by-other-PR 127/1 Mathlib.lean,Mathlib/ModelTheory/Topology/Types.lean,Mathlib/ModelTheory/Types.lean,Mathlib/Tactic/Linter/DirectoryDependency.lean 4 5 ['NoneMore', 'anishrajeev', 'github-actions', 'mathlib4-dependent-issues-bot'] fpvandoorn
assignee:fpvandoorn
19-12775
19 days ago
34-62807
34 days ago
3-63673
3 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) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-analysis 53/33 Mathlib/Analysis/Normed/Operator/Banach.lean 1 16 ['faenuccio', 'github-actions', 'kckennylau', 'leanprover-bot', 'mathlib4-merge-conflict-bot', 'themathqueen', 'yuanyi-350'] faenuccio
assignee:faenuccio
18-79034
18 days ago
116-29439
116 days ago
0-33637
9 hours
32921 faenuccio
author:faenuccio
refactor Submodule.map Following [#mathlib4 > on the definition of Submodule.map](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/on.20the.20definition.20of.20Submodule.2Emap/with/563900347) this PR refactors the definition of `Submodule.map` removing the requirement that the underlying ring homomorphism be surjective. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP awaiting-author t-algebra merge-conflict
label:t-algebra$
32/20 Mathlib/Algebra/Module/Submodule/Map.lean 1 3 ['github-actions', 'mathlib4-merge-conflict-bot'] nobody
18-77156
18 days ago
unknown
unknown
33189 peabrainiac
author:peabrainiac
feat(Geometry/Manifold): the interior of a manifold is open Show that the interior and boundary of manifolds are well-defined in the sense that the definition of interior points does not depend on a choice of chart, and conclude that the interior and boundary of manifolds are open resp. closed. We only do this for $C^1$ manifolds because while it holds for finite-dimensional topological manifolds too, it is not clear to me whether it holds for infinite-dimensional topological manifolds, so that the finite-dimensional topological case probably needs to be treated separately from this infinite-dimensional $C^1$ case anyway. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-differential-geometry awaiting-author 185/8 Mathlib/Geometry/Manifold/IsManifold/ExtChartAt.lean,Mathlib/Geometry/Manifold/IsManifold/InteriorBoundary.lean,Mathlib/Topology/Closure.lean 3 15 ['Komyyy', 'github-actions', 'grunweg', 'peabrainiac'] grunweg
assignee:grunweg
18-76232
18 days ago
23-53098
23 days ago
0-38057
10 hours
32889 artie2000
author:artie2000
feat(Algebra): forgetful lemmas for `map` and `comap` on substructures * Standardise the form of forgetful lemmas for `map` and `comap` (ie, `(co)map_toSubfoo`) * Add missing lemmas of this form * Mark all such lemmas as `simp` --- - [ ] depends on: #21031 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra awaiting-author blocked-by-other-PR merge-conflict
label:t-algebra$
72/17 Mathlib/Algebra/Algebra/NonUnitalSubalgebra.lean,Mathlib/Algebra/Algebra/Subalgebra/Basic.lean,Mathlib/Algebra/Group/Subgroup/Map.lean,Mathlib/Algebra/Module/Submodule/Map.lean,Mathlib/Algebra/Ring/Subsemiring/Basic.lean,Mathlib/Algebra/Star/Subalgebra.lean 6 30 ['YaelDillies', 'artie2000', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'vihdzp'] nobody
18-70684
18 days ago
28-46919
28 days ago
2-51242
2 days
32960 dleijnse
author:dleijnse
feat(FieldTheory): adjoin pth roots For a field `k` of exponential characteristic `p` and a subset `S` of `k`, we define the extension of `k` obtained by adjoining all `p`-th roots of elements of `S`. We prove that this is a purely inseparable extension, and provide some basic API. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra new-contributor awaiting-author
label:t-algebra$
131/0 Mathlib.lean,Mathlib/FieldTheory/PurelyInseparable/AdjoinPthRoots.lean 2 13 ['artie2000', 'chrisflav', 'dleijnse', 'erdOne', 'github-actions', 'leanprover-radar'] erdOne
assignee:erdOne
18-58228
18 days ago
18-58228
18 days ago
10-11880
10 days
33163 Aaron1011
author:Aaron1011
feat: prove subgroup of (M -> Z) is finitely generated --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-ring-theory new-contributor awaiting-author 5/0 Mathlib/RingTheory/DedekindDomain/Dvr.lean 1 2 ['erdOne', 'github-actions'] alreadydone
assignee:alreadydone
18-51178
18 days ago
18-51178
18 days ago
5-78603
5 days
33217 Blackfeather007
author:Blackfeather007
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. --- migrated from https://github.com/leanprover-community/mathlib4/pull/26857 new-contributor t-ring-theory awaiting-author 144/0 Mathlib.lean,Mathlib/RingTheory/FilteredAlgebra/AssociatedGraded.lean 2 4 ['erdOne', 'github-actions'] erdOne
assignee:erdOne
18-45519
18 days ago
18-45519
18 days ago
4-55780
4 days
32987 kim-em
author:kim-em
feat: pipeline downloads and decompression in `cache get` This PR modifies `lake exe cache get` to decompress files as they download, rather than waiting for all downloads to complete first. Previously the cache system had two sequential phases: download all files using `curl --parallel`, then decompress all files using a single `leantar` call. Now a background task spawns sequential batched `leantar` calls to decompress files as downloads complete, pipelining network I/O and disk I/O. 🤖 Prepared with Claude Code 194/30 Cache/Requests.lean 1 1 ['github-actions'] dagurtomas
assignee:dagurtomas
18-31230
18 days ago
28-32215
28 days ago
29-29019
29 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) ``` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
29/6 Mathlib/RingTheory/TensorProduct/Basic.lean 1 8 ['adomani', 'github-actions', 'kbuzzard', 'leanprover-bot', 'mathlib-bors', 'mathlib4-merge-conflict-bot'] adomani
assignee:adomani
17-64305
17 days ago
unknown
unknown
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`. More generally, this shows that given star-homomorphisms `f` and `g` from `B` to a star-algebra `A` and that the centralizer of `range g` is trivial, then `f x = U * g x * U⁻¹` for some invertible element `U` if and only if `f x = U * g x * star U` for some unitary `U`. Then a corollary to this and [AlgEquiv.eq_linearEquivConjAlgEquiv](https://leanprover-community.github.io/mathlib4_docs/Mathlib/LinearAlgebra/GeneralLinearGroup/AlgEquiv.html#AlgEquiv.eq_linearEquivConjAlgEquiv) is that star-algebra automorphisms on matrices are unitarily inner. Another quick corollary to this and [ContinuousAlgEquiv.eq_continuousLinearEquivConjContinuousAlgEquiv](https://leanprover-community.github.io/mathlib4_docs/Mathlib/Analysis/Normed/Operator/ContinuousAlgEquiv.html#ContinuousAlgEquiv.eq_continuousLinearEquivConjContinuousAlgEquiv) is that star-algebra automorphisms on endomorphisms in `ℂ`-Hilbert spaces are unitarily inner. (See #33066 for the more general version of this.) --- - [x] depends on: #28100 - [x] depends on: #28182 - [x] depends on: #28881 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-analysis awaiting-author
label:t-algebra$
138/0 Mathlib.lean,Mathlib/Analysis/Matrix/StarAlgEquiv.lean 2 5 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'themathqueen'] dagurtomas
assignee:dagurtomas
17-49361
17 days ago
17-49361
17 days ago
1-41978
1 day
33363 BoltonBailey
author:BoltonBailey
feat: add `empty_eq_image` simp lemmas Creates new simp lemmas `image_eq_empty`, similar to existing simp lemmas, but with the LHS equality reversed, so that simp can identify these when in this form. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data 7/0 Mathlib/Data/Finset/Image.lean,Mathlib/Data/Set/Image.lean 2 1 ['github-actions'] nobody
17-38073
17 days ago
17-34733
17 days ago
17-34553
17 days
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR large-import 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
17-34139
17 days ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import 227/2 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
17-33856
17 days ago
17-31509
17 days ago
64-13257
64 days
33280 michelsol
author:michelsol
feat(MeasureTheory/Integral/IntervalIntegral): add variant `integral_deriv_eq_sub_uIoo` of 2nd theorem of calculus. Add a continuous on uIcc, differentiable on uIoo, deriv version of the 2nd fundamental theorem of calculus. This corresponds to what is written [here](https://en.wikipedia.org/wiki/Fundamental_theorem_of_calculus#Second_part). For example it makes it easier to compute the integral : ```lean4 ∫ x : ℝ in 0..1, (√(1 - x ^ 2))⁻¹ = ∫ x : ℝ in 0..1, deriv arcsin x = arcsin 1 - arcsin 0 ``` It is not possible to use [`interval_deriv_eq_sub`](https://leanprover-community.github.io/mathlib4_docs/Mathlib/MeasureTheory/Integral/IntervalIntegral/FundThmCalculus.html#intervalIntegral.integral_deriv_eq_sub) which requires differentiability on all of [0,1], as `arcsin` isn't differentiable at 1. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-measure-probability new-contributor 14/0 Mathlib/MeasureTheory/Integral/IntervalIntegral/FundThmCalculus.lean 1 1 ['github-actions'] EtienneC30
assignee:EtienneC30
17-31243
17 days ago
20-55888
20 days ago
20-55708
20 days
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). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-meta 1/1 Mathlib/Tactic/GeneralizeProofs.lean 1 6 ['github-actions', 'jcommelin', 'kmill', 'mathlib4-merge-conflict-bot', 'plby'] nobody
17-27476
17 days ago
unknown
unknown
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 45 ['BoltonBailey', 'IlPreteRosso', 'TwoFX', 'github-actions', 'kckennylau', 'mathlib4-merge-conflict-bot', 'rudynicolop'] TwoFX
assignee:TwoFX
17-20161
17 days ago
26-38102
26 days ago
90-59512
90 days
25138 chrisflav
author:chrisflav
chore(RingTheory/Ideal): make `RingHom.ker` take a `RingHom` instead of `RingHomClass` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra awaiting-author merge-conflict
label:t-algebra$
317/309 Mathlib/Algebra/Algebra/Equiv.lean,Mathlib/Algebra/Algebra/Hom.lean,Mathlib/Algebra/Algebra/Hom/Rat.lean,Mathlib/Algebra/Algebra/Opposite.lean,Mathlib/Algebra/Algebra/Subalgebra/Operations.lean,Mathlib/Algebra/Algebra/Tower.lean,Mathlib/Algebra/Category/CommAlgCat/FiniteType.lean,Mathlib/Algebra/Lie/CartanExists.lean,Mathlib/Algebra/MonoidAlgebra/Basic.lean,Mathlib/Algebra/MvPolynomial/Equiv.lean,Mathlib/Algebra/MvPolynomial/Eval.lean,Mathlib/Algebra/Polynomial/AlgebraMap.lean,Mathlib/Algebra/Polynomial/Module/AEval.lean,Mathlib/Algebra/RingQuot.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Affine/Basic.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Affine/Formula.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Jacobian/Basic.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Projective/Basic.lean,Mathlib/AlgebraicGeometry/EllipticCurve/VariableChange.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Weierstrass.lean,Mathlib/AlgebraicGeometry/Pullbacks.lean,Mathlib/Combinatorics/Nullstellensatz.lean,Mathlib/FieldTheory/Minpoly/Field.lean,Mathlib/FieldTheory/PurelyInseparable/Tower.lean,Mathlib/LinearAlgebra/Semisimple.lean,Mathlib/LinearAlgebra/TensorProduct/RightExactness.lean,Mathlib/NumberTheory/NumberField/InfinitePlace/Embeddings.lean,Mathlib/RingTheory/AdicCompletion/Algebra.lean,Mathlib/RingTheory/Adjoin/Tower.lean,Mathlib/RingTheory/AdjoinRoot.lean,Mathlib/RingTheory/Algebraic/Basic.lean,Mathlib/RingTheory/Congruence/Hom.lean,Mathlib/RingTheory/Etale/Kaehler.lean,Mathlib/RingTheory/Extension/Cotangent/Basis.lean,Mathlib/RingTheory/Extension/Cotangent/LocalizationAway.lean,Mathlib/RingTheory/Extension/Generators.lean,Mathlib/RingTheory/Extension/Presentation/Basic.lean,Mathlib/RingTheory/Extension/Presentation/Core.lean,Mathlib/RingTheory/FinitePresentation.lean,Mathlib/RingTheory/FiniteStability.lean,Mathlib/RingTheory/Finiteness/NilpotentKer.lean,Mathlib/RingTheory/Ideal/Cotangent.lean,Mathlib/RingTheory/Ideal/Maps.lean,Mathlib/RingTheory/Ideal/Quotient/Operations.lean,Mathlib/RingTheory/IsAdjoinRoot.lean,Mathlib/RingTheory/Jacobson/Ring.lean,Mathlib/RingTheory/Kaehler/Basic.lean,Mathlib/RingTheory/Kaehler/JacobiZariski.lean,Mathlib/RingTheory/LocalRing/ResidueField/Fiber.lean,Mathlib/RingTheory/LocalRing/ResidueField/Ideal.lean,Mathlib/RingTheory/Localization/Algebra.lean,Mathlib/RingTheory/MvPowerSeries/Evaluation.lean,Mathlib/RingTheory/Nilpotent/Lemmas.lean,Mathlib/RingTheory/NoetherNormalization.lean,Mathlib/RingTheory/Nullstellensatz.lean,Mathlib/RingTheory/Polynomial/Basic.lean,Mathlib/RingTheory/Polynomial/UniqueFactorization.lean,Mathlib/RingTheory/Polynomial/UniversalFactorizationRing.lean,Mathlib/RingTheory/Smooth/AdicCompletion.lean,Mathlib/RingTheory/Smooth/Basic.lean,Mathlib/RingTheory/Smooth/Flat.lean,Mathlib/RingTheory/Smooth/Kaehler.lean,Mathlib/RingTheory/Smooth/NoetherianDescent.lean,Mathlib/RingTheory/Spectrum/Prime/ChevalleyComplexity.lean,Mathlib/RingTheory/Unramified/Finite.lean,Mathlib/Topology/Algebra/Module/CharacterSpace.lean,Mathlib/Topology/ContinuousMap/Ideals.lean,Mathlib/Topology/ContinuousMap/StoneWeierstrass.lean 68 8 ['chrisflav', 'erdOne', 'eric-wieser', 'github-actions', 'jcommelin', 'leanprover-community-bot-assistant', 'mathlib4-merge-conflict-bot'] nobody
17-14884
17 days ago
unknown
unknown
32865 robertmaxton42
author:robertmaxton42
(WIP) Separation axioms --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import merge-conflict 4350/12 Mathlib.lean,Mathlib/CategoryTheory/LiftingProperties/Basic.lean,Mathlib/CategoryTheory/Limits/Shapes/ConcreteCategory.lean,Mathlib/Data/Set/Basic.lean,Mathlib/Data/Set/Disjoint.lean,Mathlib/Data/Set/Image.lean,Mathlib/Data/Set/Lattice.lean,Mathlib/Data/Set/Operations.lean,Mathlib/Order/BooleanAlgebra/Set.lean,Mathlib/Topology/AlexandrovDiscrete.lean,Mathlib/Topology/Category/Lifting/Defs.lean,Mathlib/Topology/Category/Lifting/Separation.lean,Mathlib/Topology/Category/TopCat/Basic.lean,Mathlib/Topology/Category/TopCat/Limits/Basic.lean,Mathlib/Topology/Category/TopCat/Limits/Pullbacks.lean,Mathlib/Topology/Category/UProp.lean,Mathlib/Topology/Coherent.lean,Mathlib/Topology/Constructions.lean,Mathlib/Topology/ContinuousMap/Basic.lean,Mathlib/Topology/ContinuousMap/Constructions.lean,Mathlib/Topology/Inseparable.lean,Mathlib/Topology/Maps/Basic.lean,Mathlib/Topology/Order.lean,Mathlib/Topology/Order/UpperLowerSetTopology.lean,Mathlib/Topology/Separation/GDelta.lean,Mathlib/Topology/Separation/Regular.lean,Mathlib/Topology/UnitInterval.lean,Mathlib/Topology/UrysohnsLemma.lean,docs/references.bib 29 2 ['github-actions', 'mathlib4-merge-conflict-bot'] nobody
17-11954
17 days ago
unknown
unknown
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`. t-combinatorics new-contributor 76/0 Mathlib.lean,Mathlib/Combinatorics/Enumerative/RecLatticePath.lean 2 3 ['github-actions', 'mathlib4-merge-conflict-bot'] awainverse
assignee:awainverse
16-83520
16 days ago
16-82697
16 days ago
36-28736
36 days
31018 joelriou
author:joelriou
feat(CategoryTheory): the κ-accessible category of κ-directed posets WIP --- - [x] depends on: #30727 - [x] depends on: #31767 - [x] depends on: #29519 - [x] depends on: #29543 - [x] depends on: #29565 - [x] depends on: #29854 - [x] depends on: #30459 - [x] depends on: #30605 - [x] depends on: #31426 - [x] depends on: #31421 - [x] depends on: #30633 - [x] depends on: #30634 - [x] depends on: #30693 - [x] depends on: #30696 - [x] depends on: #30781 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-category-theory 446/4 Mathlib.lean,Mathlib/CategoryTheory/Presentable/Basic.lean,Mathlib/CategoryTheory/Presentable/CardinalDirectedPoset.lean,Mathlib/CategoryTheory/Presentable/SharplyLT.lean,Mathlib/Order/Category/PartOrdEmb.lean 5 4 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
16-60082
16 days ago
unknown
unknown
33386 joelriou
author:joelriou
feat(AlgebraicTopology/SimplicialSet): decidable instances --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebraic-topology WIP RFC 76/0 Mathlib.lean,Mathlib/AlgebraicTopology/SimplicialSet/Decidable.lean 2 1 ['github-actions'] nobody
16-57479
16 days ago
unknown
unknown
32688 grunweg
author:grunweg
chore: update complex analysis library overview Mathlib has the identity theorem, and also meromorphic functions. --- @kebekus I wasn't sure if there are any major results on meromorphic functions that should also be mentioned. If there are, feel free to suggest them and I will add them as well. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis 10/8 Mathlib/Analysis/Analytic/IsolatedZeros.lean,docs/overview.yaml,docs/undergrad.yaml 3 2 ['github-actions', 'kebekus'] nobody
16-36922
16 days ago
unknown
unknown
33064 DavidLedvinka
author:DavidLedvinka
feat(Probability): Add `condLExp`, conditional expectation with the Lebesgue integral Add definition of `condLExp`, conditional expectation using the Lebesgue integral. Also add basic API. t-measure-probability 275/0 Mathlib.lean,Mathlib/MeasureTheory/Function/ConditionalLExpectation.lean,Mathlib/MeasureTheory/Integral/Lebesgue/Add.lean,Mathlib/MeasureTheory/MeasurableSpace/CountablyGenerated.lean,Mathlib/MeasureTheory/MeasurableSpace/Defs.lean,Mathlib/MeasureTheory/Measure/AEMeasurable.lean 6 3 ['DavidLedvinka', 'github-actions', 'leanprover-radar'] EtienneC30
assignee:EtienneC30
16-36442
16 days ago
16-35564
16 days ago
26-38803
26 days
33143 wwylele
author:wwylele
feat(PowerSeries): pentagonal number theorem The proof is split in two files: `Mathlib/Topology/Algebra/InfiniteSum/Pentagonal.lean` for the algebraic part, and `Mathlib/RingTheory/PowerSeries/Pentagonal.lean` for the summability part. In the near future, I also plan to prove the real/complex version that branches off from the algebraic part. --- - [ ] depends on: #30436 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 324/1 Mathlib.lean,Mathlib/RingTheory/PowerSeries/Pentagonal.lean,Mathlib/Topology/Algebra/InfiniteSum/Pentagonal.lean,docs/1000.yaml 4 12 ['copilot-pull-request-reviewer', 'github-actions', 'mathlib4-dependent-issues-bot', 'vihdzp'] kex-y
assignee:kex-y
16-31261
16 days ago
18-69044
18 days ago
19-38681
19 days
33297 tb65536
author:tb65536
feat(Algebra/Polynomial/Roots): add `card_rootSet_le` This PR adds a lemma stating that `Set.ncard (p.rootSet B) ≤ p.natDegree` (we already have similar lemmas for `Polynomial.roots`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra large-import
label:t-algebra$
7/0 Mathlib/Algebra/Polynomial/Roots.lean 1 1 ['github-actions'] dagurtomas
assignee:dagurtomas
16-31260
16 days ago
20-27260
20 days ago
20-27080
20 days
33021 farmanb
author:farmanb
feat(RingTheory/IdealFilter): add ideal filters and Gabriel filters This PR introduces ideal filters on a ring and the notion of a Gabriel filter. Main additions: * `IdealFilter A`: filters on the lattice of ideals of a ring `A` * `IsUniform`: the uniformity (T1–T3) condition * `gabrielComposition` and notation `•` * `IsGabriel`: Gabriel filters (axiom T4) * A characterization `IsGabriel ↔ IsUniform ∧ F • F = F` This is preparatory infrastructure for future work relating Gabriel filters to Giraud subcategories. This development is motivated by Theorem 10.2 in Bo Stenström, *Rings and Modules of Quotients*, which identifies equivalence classes of Giraud subcategories with linear (Gabriel) topologies on a ring. The present PR provides the ring-theoretic filter infrastructure needed for that result. --- - [ ] depends on: #33390 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-ring-theory new-contributor blocked-by-other-PR 283/0 Mathlib.lean,Mathlib/RingTheory/Ideal/Colon.lean,Mathlib/RingTheory/IdealFilter/Basic.lean,docs/references.bib 4 21 ['erdOne', 'farmanb', 'github-actions', 'mathlib4-dependent-issues-bot'] mattrobball
assignee:mattrobball
15-63489
15 days ago
15-63490
15 days ago
11-73862
11 days
24665 Komyyy
author:Komyyy
feat(Mathlib/Topology/Metrizable/Uniformity): every uniform space is generated by a family of pseudometrics --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-topology merge-conflict 54/0 Mathlib/Topology/Metrizable/Uniformity.lean 1 2 ['github-actions', 'mathlib4-merge-conflict-bot'] nobody
15-44008
15 days ago
unknown
unknown
33406 dupuisf
author:dupuisf
feat: add basics of majorization This PR defines [majorization](https://en.wikipedia.org/wiki/Majorization). This is needed to develop the theory of unitarily invariant norms on `ℂ^n`, in particular Schatten norms. --- - [ ] depends on: #33394 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR 784/15 Mathlib.lean,Mathlib/Analysis/Convex/DoublyStochasticMatrix.lean,Mathlib/Analysis/Convex/Majorization/Basic.lean,Mathlib/Analysis/Convex/Majorization/Defs.lean,Mathlib/Data/Finset/BooleanAlgebra.lean,Mathlib/Data/Finset/Card.lean,Mathlib/Data/Finset/Image.lean,Mathlib/Data/Finset/Max.lean,Mathlib/Data/Finset/Powerset.lean,Mathlib/Data/Fintype/Card.lean,Mathlib/Order/Interval/Finset/Fin.lean 11 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
15-19472
15 days ago
unknown
unknown
33381 urkud
author:urkud
feat: add a version of the Schwarz lemma Add a version of the Schwarz lemma that is midway between the original lemma and Pick's version. Use it to show that a function that is separately holomorphic on a polydisc and is bounded on this polydisc must be continuous on it. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) - [ ] depends on: #33368 - [x] depends on: #33362 t-analysis blocked-by-other-PR merge-conflict 475/91 Mathlib.lean,Mathlib/Analysis/Complex/Schwarz.lean,Mathlib/Analysis/Complex/UnitDisc/Basic.lean,Mathlib/Analysis/Complex/UnitDisc/Schwarz.lean,Mathlib/Analysis/Complex/UnitDisc/Shift.lean 5 22 ['girving', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'urkud'] nobody
15-14717
15 days ago
16-69597
16 days ago
0-38
38 seconds
33080 sinhp
author:sinhp
feat(Category Theory): Cartesian Natural Transformation This PR defines cartesian natural transformations between functors and proves they are closed under horizontal and vertical composition. Also we prove the following results: - `NatTrans.isCartesian_of_discrete` shows that any natural transformation between functors from a discrete category is cartesian. - `NatTrans.isCartesian_of_isIso` shows that any natural isomorphism is cartesian. - `NatTrans.isIso_of_isCartesian_of_isIso_app_terminal` shows that a cartesian natural transformation is an isomorphism if its component at a terminal object is an isomorphism. - `NatTrans.isCartesian_of_isPullback_isTerminal_from` shows that a natural transformation is cartesian if all its naturality squares to the terminal object are pullback squares. This material is adapted from the polynomial functors project developed during the Trimester "Prospects of Formal Mathematics" at the Hausdorff Institute (HIM) in Bonn: https://github.com/sinhp/Poly Co-authored-by: Wojciech Nawrocki --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory awaiting-author 145/0 Mathlib.lean,Mathlib/CategoryTheory/NatTransCartesian.lean 2 7 ['dagurtomas', 'github-actions', 'joelriou', 'sinhp'] nobody
14-62118
14 days ago
14-62118
14 days ago
3-19604
3 days
33394 dupuisf
author:dupuisf
feat: add lemmas about doubly stochastic matrices This PR adds a few basic lemmas about doubly stochastic matrices. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis awaiting-author 59/0 Mathlib/Analysis/Convex/DoublyStochasticMatrix.lean 1 3 ['dupuisf', 'github-actions', 'j-loreaux'] nobody
14-55120
14 days ago
14-59867
14 days ago
1-51881
1 day
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP awaiting-bench t-algebra blocked-by-other-PR merge-conflict
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
14-7297
14 days ago
unknown
unknown
33448 astrainfinita
author:astrainfinita
refactor: deprecate `ContinuousLinearMapClass` This PR continues the work from #18748. Original PR: https://github.com/leanprover-community/mathlib4/pull/18748 t-topology t-algebra awaiting-author
label:t-algebra$
55/41 Mathlib/Analysis/CStarAlgebra/PositiveLinearMap.lean,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/CharacterSpace.lean,Mathlib/Topology/Algebra/Module/Equiv.lean,Mathlib/Topology/Algebra/Module/FiniteDimension.lean,Mathlib/Topology/Algebra/Module/LinearMap.lean,Mathlib/Topology/Algebra/Module/StrongTopology.lean,Mathlib/Topology/Algebra/Module/WeakDual.lean 11 10 ['Ruben-VandeVelde', 'astrainfinita', 'github-actions', 'leanprover-radar'] nobody
13-81321
13 days ago
13-81321
13 days ago
0-14664
4 hours
21031 YaelDillies
author:YaelDillies
chore: get rid of generic hom coercions --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP 168/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 17 ['Vierkantor', 'YaelDillies', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-merge-conflict-bot', 'urkud'] Vierkantor
assignee:Vierkantor
13-57996
13 days ago
unknown
unknown
33462 eric-wieser
author:eric-wieser
feat: teach `fun_prop` about `ContinousMultilinearMap.compContinuousLinearMap` For now I've omitted the curried version --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis 46/0 Mathlib/Analysis/Normed/Module/Multilinear/Basic.lean 1 3 ['github-actions', 'sgouezel'] nobody
13-45045
13 days ago
unknown
unknown
32803 erdOne
author:erdOne
feat(RIngTheory): more-linear version of `tensorKaehlerEquiv` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-ring-theory 83/7 Mathlib/RingTheory/Kaehler/TensorProduct.lean 1 16 ['Ruben-VandeVelde', 'erdOne', 'github-actions', 'mattrobball', 'robin-carlier'] mattrobball
assignee:mattrobball
13-39561
13 days ago
13-38819
13 days ago
23-20482
23 days
32725 joelriou
author:joelriou
feat(CategoryTheory): presheaves of types which preserve a limit Let `F : J ⥤ Cᵒᵖ` be a functor. We show that a presheaf `P : Cᵒᵖ ⥤ Type w` preserves the limit of `F` iff `P` is a local object with respect to a suitable family of morphisms in `Cᵒᵖ ⥤ Type w` (this family contains `1` or `0` morphism depending on whether the limit of `F` exists or not). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory awaiting-author 187/0 Mathlib.lean,Mathlib/CategoryTheory/MorphismProperty/Basic.lean,Mathlib/CategoryTheory/MorphismProperty/IsSmall.lean,Mathlib/CategoryTheory/ObjectProperty/FunctorCategory/Presheaf.lean,Mathlib/CategoryTheory/ObjectProperty/Local.lean 5 6 ['github-actions', 'joelriou', 'robin-carlier'] nobody
13-1878
13 days ago
13-1878
13 days ago
3-75996
3 days
32840 joelriou
author:joelriou
chore(CategoryTheory): remove the old Ext API As it is now possible to compute `Ext`-groups (defined using the derived category) using an injective resolution #32105 or a projective resolution #32816, the old `Ext` API (based on left derived functors) is removed. WIP (more API for the new `Ext` is necessary...) --- - [ ] depends on: #32816 - [ ] depends on: #32105 - [ ] depends on: #32814 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) file-removed t-category-theory large-import merge-conflict WIP 546/116 Mathlib.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/Linear.lean,Mathlib/Algebra/Homology/DerivedCategory/KInjective.lean,Mathlib/Algebra/Homology/DerivedCategory/KProjective.lean,Mathlib/Algebra/Homology/Embedding/IsSupported.lean,Mathlib/Algebra/Homology/LocalCohomology.lean,Mathlib/CategoryTheory/Abelian/Ext.lean,Mathlib/CategoryTheory/Abelian/Injective/Ext.lean,Mathlib/CategoryTheory/Abelian/Injective/Extend.lean,Mathlib/CategoryTheory/Abelian/Projective/Ext.lean,Mathlib/CategoryTheory/Abelian/Projective/Extend.lean,Mathlib/RepresentationTheory/Homological/Resolution.lean 12 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
12-82339
12 days ago
unknown
unknown
33133 0xTerencePrime
author:0xTerencePrime
feat(Algebra/Group/Center): add Decidable (IsMulCentral a) instance This PR adds a `Decidable` instance for `IsMulCentral a`. ### Summary The structure `IsMulCentral` was missing a `Decidable` instance. This PR provides the instance by leveraging `isMulCentral_iff`, enabling decidability for both multiplicative and additive (via `to_additive`) structures. ### Verification - `lake build Mathlib.Algebra.Group.Center` passed. - `lake exe runLinter Mathlib.Algebra.Group.Center` passed. t-algebra new-contributor awaiting-author
label:t-algebra$
7/0 Mathlib/Algebra/Group/Center.lean 1 3 ['github-actions', 'robin-carlier'] ocfnash
assignee:ocfnash
12-79369
12 days ago
12-79369
12 days ago
12-58151
12 days
33276 NicolaBernini
author:NicolaBernini
feat: Rename List.reverse_perm to List.reverse_perm_self and List.reverse_perm' to List.reverse_perm_iff --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor awaiting-author 17/15 Mathlib/Algebra/BigOperators/Group/List/Basic.lean,Mathlib/Data/Finset/Dedup.lean,Mathlib/Data/List/Basic.lean,Mathlib/Data/List/Defs.lean,Mathlib/Data/List/Perm/Lattice.lean,Mathlib/Data/List/Permutation.lean,Mathlib/Data/Multiset/Defs.lean,Mathlib/NumberTheory/Divisors.lean 8 4 ['Ruben-VandeVelde', 'github-actions'] kim-em
assignee:kim-em
12-68503
12 days ago
16-78697
16 days ago
3-79472
3 days
33351 themathqueen
author:themathqueen
chore(Analysis/LocallyConvex/SeparatingDual): generalize `Algebra.IsCentral.instContinuousLinearMap` ... to two different scalar fields. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis awaiting-author 35/22 Mathlib/Analysis/LocallyConvex/SeparatingDual.lean,Mathlib/Topology/Algebra/Module/LinearMap.lean 2 7 ['github-actions', 'j-loreaux', 'leanprover-radar', 'themathqueen'] nobody
12-48479
12 days ago
14-59382
14 days ago
3-45787
3 days
33191 sinhp
author:sinhp
feat(CategoryTheory): Locally cartesian closed structure on presheaf categories The category of presheaves on a small category `C` is locally cartesian closed. --- - [ ] depends on: #30375 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-category-theory blocked-by-other-PR merge-conflict 703/0 Mathlib.lean,Mathlib/CategoryTheory/LocallyCartesianClosed/Basic.lean,Mathlib/CategoryTheory/LocallyCartesianClosed/ChosenPullbacksAlong.lean,Mathlib/CategoryTheory/LocallyCartesianClosed/ExponentiableMorphism.lean,Mathlib/CategoryTheory/LocallyCartesianClosed/Sections.lean 5 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
12-46313
12 days ago
unknown
unknown
33495 vihdzp
author:vihdzp
chore(RingTheory/HahnSeries/Basic): redefine `order` using `unbotD` --- - [ ] depends on: #33494 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-ring-theory blocked-by-other-PR 67/26 Mathlib/RingTheory/HahnSeries/Basic.lean 1 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
12-34221
12 days ago
unknown
unknown
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-meta 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'] nobody
12-29947
12 days ago
99-65366
99 days ago
58-76266
58 days
25500 eric-wieser
author:eric-wieser
feat: delaborators for metadata Being able to see these is very important when debugging tactic failures. Probably these could be upstreamed, but I don't think that's a reason not to merge them here first. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import merge-conflict awaiting-author delegated t-meta 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'] nobody
12-29899
12 days ago
139-60412
139 days ago
42-79607
42 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) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-meta 16/0 Mathlib/Tactic/FunProp.lean 1 6 ['Vierkantor', 'github-actions', 'grunweg', 'kckennylau', 'mathlib4-merge-conflict-bot'] nobody
12-29885
12 days ago
99-69082
99 days ago
57-61561
57 days
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-algebraic-geometry 66/0 Mathlib/AlgebraicGeometry/ProjectiveSpectrum/Basic.lean 1 4 ['github-actions', 'jcommelin'] nobody
12-29857
12 days ago
51-78173
51 days ago
44-11265
44 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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta awaiting-author 63/5 Mathlib/Lean/Message.lean 1 20 ['adomani', 'github-actions', 'grunweg', 'mathlib4-merge-conflict-bot', 'thorimur'] nobody
12-29845
12 days ago
40-54828
40 days ago
20-86334
20 days
27262 Timeroot
author:Timeroot
feat(Tactic/Bound): bound? for proof scripts --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-meta 22/7 Mathlib/Tactic/Bound.lean 1 13 ['JovanGerb', 'Timeroot', 'github-actions', 'j-loreaux', 'mathlib4-merge-conflict-bot'] nobody
12-21809
12 days ago
104-34134
104 days ago
9-17828
9 days
30758 Timeroot
author:Timeroot
chore: tag abs_inv and abs_div with grind= --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
4/3 Mathlib/Algebra/Order/Field/Basic.lean,Mathlib/Algebra/Order/Ring/Abs.lean 2 2 ['Timeroot', 'Vierkantor', 'github-actions'] kim-em
assignee:kim-em
12-20698
12 days ago
41-61511
41 days ago
43-73485
43 days
33481 NoneMore
author:NoneMore
feat(ModelTheory/Encoding): add `Countable` instances for (bounded) formulas in countable languages Prepare for the OTT proof. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-logic new-contributor 27/0 Mathlib/ModelTheory/Encoding.lean 1 1 ['github-actions'] nobody
12-15015
12 days ago
12-14079
12 days ago
12-81800
12 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
label:t-algebra$
188/0 Mathlib.lean,Mathlib/Algebra/Homology/EulerCharacteristic.lean 2 10 ['github-actions', 'jessealama', 'joelriou', 'mathlib4-merge-conflict-bot'] mattrobball
assignee:mattrobball
12-7895
12 days ago
12-7020
12 days ago
27-19996
27 days
33256 joelriou
author:joelriou
feat(CategoryTheory/Sites): characterization of (pre)stacks for a precoverage When a precoverage `J` satisfies slightly stronger axioms than those of pretopologies, then in order to verify that a pseudofunctor is a prestack (resp. a stack), it suffices to check that the `toDescentData` functors attached to presieves in `J` are fully faithful (resp. equivalences). This is a draft... --- - [ ] depends on: #33518 - [x] depends on: #33287 - [x] depends on: #33179 - [x] depends on: #33195 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-category-theory blocked-by-other-PR 438/1 Mathlib.lean,Mathlib/CategoryTheory/Sites/Descent/DescentData.lean,Mathlib/CategoryTheory/Sites/Descent/Precoverage.lean,Mathlib/CategoryTheory/Sites/PrecoverageToGrothendieck.lean,Mathlib/CategoryTheory/Sites/Sieves.lean 5 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
12-417
12 days ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis awaiting-author 120/0 Mathlib/Analysis/SpecialFunctions/Trigonometric/Basic.lean 1 11 ['LLaurance', 'artie2000', 'github-actions', 'j-loreaux'] nobody
11-86092
11 days ago
27-46423
27 days ago
15-35949
15 days
32654 YaelDillies
author:YaelDillies
feat(Combinatorics): a clique has size at most the chromatic number There already exists a version of this lemma for cliques given by a set, but it's impractical to provide an explicit clique on an explicit graph as a set, rather than an indexed family, especially because computing the size of the set would then involve proving that it is the range of an injective function, even though being a clique already implies being injective! Application: google-deepmind/formal-conjectures#1369 Also rename `coloringOfIsEmpty` and `colorable_of_isEmpty` to leverage anonymous dot notation, and make more arguments implicit. From FormalConjectures --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics 51/40 Mathlib/Combinatorics/SimpleGraph/Basic.lean,Mathlib/Combinatorics/SimpleGraph/Coloring.lean 2 20 ['SnirBroshi', 'YaelDillies', 'github-actions'] b-mehta
assignee:b-mehta
11-83106
11 days ago
11-82290
11 days ago
36-56332
36 days
33520 NoneMore
author:NoneMore
feat(ModelTheory/ElementarySubstructures): add a variant of Tarski-Vaught test taking sets as input There should exist an `ElementarySubstructure.copy` such that we can directly bundle the set itself instaed of its closure as an elementary substructure. The other direction depends on #33458. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-logic new-contributor 63/0 Mathlib/ModelTheory/ElementarySubstructures.lean 1 1 ['github-actions'] nobody
11-68454
11 days ago
11-79857
11 days ago
11-79677
11 days
33463 khwilson
author:khwilson
feat(Mathlib/Analysis/Polynomial/MahlerMeasure): Mahler Measure for other rings Define `mahlerMeasure'` which allows you specify a norm preserving map `v` from any `NormedRing A` (or more general) to `ℂ`. Also provide wrappers around the main `mahlerMeasure` lemmas that are used for estimation. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor 96/2 Mathlib/Analysis/Polynomial/MahlerMeasure.lean,Mathlib/NumberTheory/MahlerMeasure.lean 2 16 ['github-actions', 'khwilson', 'plp127', 'vlad902'] nobody
11-64316
11 days ago
unknown
unknown
33514 urkud
author:urkud
feat(Analysis/../Connected): balls are preconnected --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis awaiting-author 6/0 Mathlib/Analysis/Normed/Module/Connected.lean 1 3 ['github-actions', 'sgouezel', 'urkud'] nobody
11-61233
11 days ago
11-76000
11 days ago
0-19965
5 hours
32608 PrParadoxy
author:PrParadoxy
feat(LinearAlgebra/PiTensorProduct): API for PiTensorProducts indexed by sets This PR addresses a TODO item in LinearAlgebra/PiTensorProduct.lean: * API for the various ways ι can be split into subsets; connect this with the binary tensor product -- specifically by describing tensors of type ⨂ (i : S), M i, for S : Set ι. Our primary motivation is to formalise the notion of "restricted tensor products". This will be the content of a follow-up PR. Beyond that, the Set API is natural in contexts where the index type has an independent interpretation. An example is quantum physics, where ι ranges over distinguishable degrees of freedom, and where its is common practice to annotate objects by the set of indices they are defined on. --- Stub file with preliminary definition of the restricted tensor product as a direct limit of tensors indexed by finite subsets of an index type: https://github.com/PrParadoxy/mathlib4/blob/restricted-stub/Mathlib/LinearAlgebra/PiTensorProduct/Restricted.lean --- - [x] depends on: #32598 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor awaiting-zulip 300/2 Mathlib.lean,Mathlib/LinearAlgebra/PiTensorProduct.lean,Mathlib/LinearAlgebra/PiTensorProduct/Set.lean 3 28 ['PrParadoxy', 'dagurtomas', 'eric-wieser', 'github-actions', 'goliath-klein', 'leanprover-radar', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] dagurtomas
assignee:dagurtomas
11-59342
11 days ago
23-59045
23 days ago
10-63624
10 days
33502 MrQubo
author:MrQubo
fix(Tactic/ProxyType): Pass params explicitly in proxy_equiv% implementation Fix [#mathlib4 > `deriving Fintype` with Prop](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/.60deriving.20Fintype.60.20with.20Prop/with/566118621) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-meta WIP 12/2 Mathlib/Tactic/ProxyType.lean,MathlibTest/DeriveFintype.lean 2 7 ['MrQubo', 'github-actions', 'kmill'] kmill
assignee:kmill
11-46293
11 days ago
11-46294
11 days ago
0-57325
15 hours
22657 Xmask19
author:Xmask19
feat: a graph is maximally acyclic iff it is a tree --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-combinatorics new-contributor 86/0 Mathlib/Combinatorics/SimpleGraph/Acyclic.lean 1 8 ['Rida-Hamadani', 'SnirBroshi', 'b-mehta', 'github-actions', 'grunweg', 'mathlib4-merge-conflict-bot'] b-mehta
assignee:b-mehta
11-39386
11 days ago
unknown
unknown
33416 vihdzp
author:vihdzp
chore(Order/GameAdd): add `elab_as_elim` attributes This PR does three things: - Rename `GameAdd.fix` to the more illustrative `GameAdd.recursion` - Add `elab_as_elim` attributes on `GameAdd.recursion` - Deprecate the duplicate `GameAdd.induction` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order 24/14 Mathlib/Order/GameAdd.lean,Mathlib/SetTheory/PGame/Order.lean,Mathlib/SetTheory/ZFC/Ordinal.lean 3 1 ['github-actions'] Vierkantor
assignee:Vierkantor
11-31239
11 days ago
15-28383
15 days ago
15-28203
15 days
33475 BoltonBailey
author:BoltonBailey
feat(Logic/IsEmpty): add theorems relating surjectivity and emptiness In particular, this adds a lemma saying that with an empty domain, a function is surjective iff its range is empty, and various forms of this. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-logic 11/2 Mathlib/Logic/IsEmpty.lean 1 13 ['BoltonBailey', 'SnirBroshi', 'eric-wieser', 'github-actions'] nobody
11-3216
11 days ago
10-85801
10 days ago
13-10412
13 days
33247 sun123zxy
author:sun123zxy
feat(Mathlib/RingTheory/Ideal/Cotangent): dimension of cotangent spaces It is shown that the span rank of the maximal ideal of a local ring equals the dimension of the cotangent space if the maximal ideal is finitely generated. To avoid unnecessary imports, the original `Mathlib/RingTheory/Nakayama` is now moved to `Mathlib/RingTheory/Nakayama/Basic`. --- - [ ] depends on: #33359 - [ ] depends on: #33361 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) file-removed new-contributor t-ring-theory blocked-by-other-PR WIP merge-conflict 314/20 Mathlib.lean,Mathlib/Algebra/Module/SpanRank.lean,Mathlib/RingTheory/Ideal/Cotangent.lean,Mathlib/RingTheory/Ideal/KrullsHeightTheorem.lean,Mathlib/RingTheory/LocalRing/Module.lean,Mathlib/RingTheory/LocalRing/Quotient.lean,Mathlib/RingTheory/Nakayama/Basic.lean,Mathlib/RingTheory/Nakayama/SpanRank.lean,Mathlib/RingTheory/Regular/RegularSequence.lean,Mathlib/RingTheory/Support.lean 10 11 ['erdOne', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'sun123zxy'] nobody
10-78801
10 days ago
18-45837
18 days ago
3-69477
3 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). [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-ring-theory 81/0 Mathlib.lean,Mathlib/RingTheory/TwoSidedIdeal/SpanAsSum.lean 2 7 ['github-actions', 'kckennylau', 'mathlib4-merge-conflict-bot'] YaelDillies
assignee:YaelDillies
10-77545
10 days ago
167-12527
167 days ago
35-41733
35 days
30927 callesonne
author:callesonne
feat(Bicategory/Yoneda): add the yoneda pseudofunctor --- - [ ] depends on: #30926 - [x] depends on: #30895 - [x] depends on: #25901 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 81/3 Mathlib.lean,Mathlib/CategoryTheory/Bicategory/Basic.lean,Mathlib/CategoryTheory/Bicategory/Yoneda.lean,Mathlib/CategoryTheory/Category/Cat.lean,Mathlib/Data/Opposite.lean 5 4 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
10-77542
10 days ago
unknown
unknown
33479 zcyemi
author:zcyemi
feat(Geometry/Euclidean/Angle/Sphere): Add theorem about cospherical points on two intersecting lines --- Add `cospherical_of_mul_dist_eq_mul_dist_of_angle_eq_pi`. This theorem is the converse of `EuclideanGeometry.mul_dist_eq_mul_dist_of_cospherical_of_angle_eq_pi`. However, the ambient type is required to be two-dimensional, i.e. `Fact (finrank ℝ V = 2)`. I don‘t think (not entirely sure) that lifting the ambient space from dimension 2 to arbitrary dimension is reasonable for this theorem, since the proof is entirely carried out in a two-dimensional plane. Therefore, I place this theorem in `Euclidean/Angle/Sphere` rather than `Euclidean/Sphere/Power`. Deps: - [ ] depends on: #33365 t-euclidean-geometry awaiting-author 69/0 Mathlib/Geometry/Euclidean/Angle/Oriented/Affine.lean,Mathlib/Geometry/Euclidean/Angle/Sphere.lean 2 4 ['github-actions', 'jsm28', 'mathlib4-dependent-issues-bot'] nobody
10-76682
10 days ago
unknown
unknown
33375 kex-y
author:kex-y
feat(Probability): Local and stable properties --- Defines local and stable properties which is useful for local martingales. - [x] depends on: #33371 - [x] depends on: #33374 - [ ] depends on: #33372 Co-authored-by: @RemyDegenne [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) brownian t-measure-probability blocked-by-other-PR 477/0 Mathlib/Probability/Process/LocalProperty.lean,Mathlib/Probability/Process/Stopping.lean 2 4 ['github-actions', 'kex-y', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
10-68803
10 days ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-analysis 146/0 Mathlib.lean,Mathlib/Analysis/Complex/BorelCaratheodory.lean,docs/1000.yaml 3 5 ['Ruben-VandeVelde', 'github-actions', 'grunweg', 'maksym-radziwill', 'mathlib4-merge-conflict-bot'] nobody
10-57054
10 days ago
59-4340
59 days ago
0-31904
8 hours
28013 astrainfinita
author:astrainfinita
feat: Lindemann-Weierstrass Theorem This PR continues the work from #6718. -------- - [x] depends on: #18693 - [x] depends on: #29121 t-algebra t-analysis awaiting-author merge-conflict
label:t-algebra$
1106/55 Mathlib.lean,Mathlib/Algebra/MonoidAlgebra/Basic.lean,Mathlib/Algebra/MonoidAlgebra/MapDomain.lean,Mathlib/Algebra/Polynomial/Factors.lean,Mathlib/Data/Finsupp/Defs.lean,Mathlib/Data/Finsupp/Indicator.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 12 15 ['astrainfinita', 'github-actions', 'grunweg', 'j-loreaux', 'jcommelin', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
10-46700
10 days ago
59-43307
59 days ago
3-85209
3 days
32886 alreadydone
author:alreadydone
refactor(Algebra/Order): change `MulArchimedeanClass.subgroup` to `FiniteArchimedeanClass.subgroup` This gets rid of a junk value without much modification the main HahnEmbedding application. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-order
label:t-algebra$
298/157 Mathlib/Algebra/Order/Archimedean/Class.lean,Mathlib/Algebra/Order/Module/Archimedean.lean,Mathlib/Algebra/Order/Module/HahnEmbedding.lean 3 7 ['alreadydone', 'github-actions', 'vihdzp', 'wwylele'] Vierkantor
assignee:Vierkantor
10-43661
10 days ago
10-42788
10 days ago
31-22910
31 days
31361 alreadydone
author:alreadydone
feat(Algebra/Order): convex subgroups --- - [ ] depends on: #32886 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-order blocked-by-other-PR merge-conflict
label:t-algebra$
408/0 Mathlib.lean,Mathlib/Algebra/Order/Archimedean/Class.lean,Mathlib/Algebra/Order/Group/Convex.lean,Mathlib/Order/Birkhoff.lean,Mathlib/Order/Quotient.lean 5 23 ['alreadydone', 'github-actions', 'kckennylau', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'vihdzp', 'wwylele'] Vierkantor
assignee:Vierkantor
10-43356
10 days ago
31-27898
31 days ago
4-39793
4 days
21344 kbuzzard
author:kbuzzard
chore: attempt to avoid diamond in OreLocalization --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) please-adopt t-algebra
label:t-algebra$
16/5 Mathlib/RingTheory/OreLocalization/Basic.lean 1 6 ['erdOne', 'github-actions', 'kbuzzard'] nobody
10-41876
10 days ago
unknown
unknown
33112 alreadydone
author:alreadydone
feat(GroupAction): `(M →[M] M) ≃* Mᵐᵒᵖ` This comes up in #33108 in the form that permutations of a group commuting with the left multiplications are the right multiplications. The Semiring versions are already in mathlib. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-group-theory awaiting-author
label:t-algebra$
41/3 Mathlib/GroupTheory/GroupAction/Hom.lean 1 2 ['github-actions', 'robin-carlier'] mattrobball
assignee:mattrobball
10-38720
10 days ago
12-74573
12 days ago
13-49136
13 days
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR t-euclidean-geometry 485/56 Mathlib.lean,Mathlib/Geometry/Euclidean/Angle/Bisector.lean,Mathlib/Geometry/Euclidean/Angle/Incenter.lean,Mathlib/Geometry/Euclidean/Projection.lean 4 4 ['github-actions', 'jsm28', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
10-32417
10 days ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-euclidean-geometry blocked-by-other-PR 1105/56 Mathlib.lean,Mathlib/Analysis/Convex/Side.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 8 6 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
10-32413
10 days 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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-euclidean-geometry blocked-by-other-PR 873/56 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 5 ['github-actions', 'jsm28', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'peakpoint'] nobody
10-32400
10 days ago
unknown
unknown
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π. Existing lemmas have hypotheses of the form `(hp' : p' ∈ s₁ ⊓ s₂)` changed to `(hp'₁ : p' ∈ s₁) (hp'₂ : p' ∈ s₂)`, matching new lemmas, on the basis that the natural way to prove the first form is to use proofs of the two separate hypotheses. --- - [ ] depends on: #30474 - [ ] depends on: #30477 - [ ] depends on: #30600 - [ ] depends on: #30703 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-euclidean-geometry 207/56 Mathlib/Geometry/Euclidean/Angle/Bisector.lean,Mathlib/Geometry/Euclidean/Projection.lean 2 27 ['JovanGerb', 'eric-wieser', 'github-actions', 'jsm28', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] JovanGerb
assignee:JovanGerb
10-32336
10 days ago
26-30664
26 days ago
61-28585
61 days
33467 euprunin
author:euprunin
chore: golf using `grind`. add `grind` annotations. --- The goal of this golfing PR is to decrease the number of times lemmas are called explicitly (replacing calls to lemmas with calls to tactics). Any decrease in compilation time is a welcome side effect, although it is not a primary objective. Trace profiling results (shown if ≥10 ms before or after): * `CategoryTheory.Limits.Pi.ι_π`: <10 ms before, 40 ms after * `CategoryTheory.Limits.Sigma.ι_π`: <10 ms before, 39 ms after * `Stream'.Seq.head_eq_none_iff`: <10 ms before, 87 ms after * `Part.mem_ωSup`: 37 ms before, <10 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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 10/24 Mathlib/CategoryTheory/EqToHom.lean,Mathlib/CategoryTheory/Limits/Shapes/ZeroMorphisms.lean,Mathlib/Data/Seq/Defs.lean,Mathlib/Order/OmegaCompletePartialOrder.lean 4 3 ['euprunin', 'github-actions', 'leanprover-radar'] alexjbest
assignee:alexjbest
10-31234
10 days ago
13-37121
13 days ago
13-36941
13 days
33469 erdOne
author:erdOne
feat(LinearAlgebra): make TensorProduct.finsuppLeft and friends heterobasic --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 77/137 Mathlib/LinearAlgebra/DirectSum/Finsupp.lean,Mathlib/LinearAlgebra/DirectSum/TensorProduct.lean,Mathlib/LinearAlgebra/TensorProduct/Basis.lean,Mathlib/LinearAlgebra/TensorProduct/Submodule.lean,Mathlib/RepresentationTheory/Coinvariants.lean,Mathlib/RepresentationTheory/Rep.lean,Mathlib/RingTheory/Flat/FaithfullyFlat/Basic.lean,Mathlib/RingTheory/Ideal/Quotient/Index.lean,Mathlib/RingTheory/LocalRing/Module.lean,Mathlib/RingTheory/Localization/BaseChange.lean,Mathlib/RingTheory/PicardGroup.lean,Mathlib/RingTheory/TensorProduct/IsBaseChangeFree.lean,Mathlib/RingTheory/TensorProduct/MvPolynomial.lean 13 1 ['github-actions'] mariainesdff
assignee:mariainesdff
10-31233
10 days ago
13-33944
13 days ago
13-33764
13 days
33470 erdOne
author:erdOne
feat: generalize `Polynomial.freeMonic` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 80/52 Mathlib.lean,Mathlib/Algebra/Polynomial/FreeMonic.lean,Mathlib/RingTheory/Polynomial/UniversalFactorizationRing.lean 3 1 ['github-actions'] thorimur
assignee:thorimur
10-31233
10 days ago
13-39501
13 days ago
13-39321
13 days
33364 BoltonBailey
author:BoltonBailey
feat(Analysis/Convex/SimplicialComplex): add AbstractSimplicialComplex + constructions This adds the concept of [abstract simplicial complex](https://en.wikipedia.org/wiki/Abstract_simplicial_complex) (and refactors SimplicialComplex in terms of it. It also adds constructions that makes it easy to define a simplicial complex for any index family of points which is downward closed and which is affinely independent. I also include a construction of (abstract and geometric) simplicial complexes associated with a SimpleGraph, where vertices become 0-faces and edges become 1-faces, which could be useful later in defining the topological notion of a graph embedding. Co-authored-by: Claude Opus 4.5 --- Notes: Perhaps it would be better to use stdSimplex as the underlying space for the graph? [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis WIP t-algebraic-topology awaiting-author 289/14 Mathlib.lean,Mathlib/AlgebraicTopology/SimplicialComplex/Basic.lean,Mathlib/Analysis/Convex/SimplicialComplex/AffineIndependentUnion.lean,Mathlib/Analysis/Convex/SimplicialComplex/Basic.lean,Mathlib/LinearAlgebra/AffineSpace/Independent.lean 5 11 ['BoltonBailey', 'github-actions', 'peabrainiac'] nobody
10-31001
10 days ago
15-43009
15 days ago
0-76618
21 hours
33039 euprunin
author:euprunin
chore(Data/List): deprecate `ext_get_iff` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data 1/7 Mathlib/Data/List/Basic.lean 1 5 ['euprunin', 'github-actions', 'jcommelin'] pechersky
assignee:pechersky
9-83128
9 days ago
20-41964
20 days ago
21-18888
21 days
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). --- - [x] depends on: #30089 WIP t-number-theory 242/25 Mathlib.lean,Mathlib/NumberTheory/LSeries/AbstractFuncEq.lean,Mathlib/NumberTheory/LSeries/HurwitzZetaOdd.lean,Mathlib/NumberTheory/ModularForms/LFunction.lean 4 7 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
9-74514
9 days ago
unknown
unknown
32978 archiebrowne
author:archiebrowne
feat(NumberTheory/ModularForms/Basic): Provide definition of the products of finitely many modular forms `finprod_equal_weights`: the product of n modular forms of weight k is a modular form of weight n * k `inprod_add_weights`: the product of n modular forms of different weights has weight the sum of the weights new-contributor t-number-theory awaiting-author 97/18 Mathlib/NumberTheory/ModularForms/Basic.lean,Mathlib/NumberTheory/ModularForms/NormTrace.lean,Mathlib/NumberTheory/ModularForms/SlashActions.lean,Mathlib/NumberTheory/ModularForms/SlashInvariantForms.lean,Mathlib/Order/Filter/ZeroAndBoundedAtFilter.lean 5 19 ['archiebrowne', 'github-actions', 'loefflerd', 'wwylele'] loefflerd
assignee:loefflerd
9-74211
9 days ago
27-1679
27 days ago
2-44108
2 days
33601 nielstron
author:nielstron
feat(Computability/ContextFreeGrammar): Concatenation of CFGs is CFG --- - [ ] depends on: #33599 - [ ] depends on: #33592 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-computability new-contributor blocked-by-other-PR 946/0 Mathlib/Computability/ContextFreeGrammar.lean 1 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
9-71660
9 days ago
unknown
unknown
29624 mcdoll
author:mcdoll
feat(LinearAlgebra/LinearPMap): add definition of resolvent and first resolvent identity --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-analysis awaiting-author
label:t-algebra$
189/9 Mathlib/LinearAlgebra/LinearPMap.lean 1 10 ['github-actions', 'j-loreaux', 'mathlib4-merge-conflict-bot', 'mcdoll'] kim-em
assignee:kim-em
9-69993
9 days ago
50-26690
50 days ago
64-58845
64 days
33599 nielstron
author:nielstron
feat(Computability/ContextFreeGrammar): closure under union --- This PR picks up https://github.com/leanprover-community/mathlib4/pull/13514 and resolves the outstanding errors. - [ ] depends on #33592 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-computability new-contributor 506/0 Mathlib/Computability/ContextFreeGrammar.lean 1 1 ['github-actions'] nobody
9-65133
9 days ago
9-71029
9 days ago
9-70849
9 days
30375 sinhp
author:sinhp
feat(CategoryTheory): Basics of Locally Cartesian Closed Categories Supersedes 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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory merge-conflict 703/0 Mathlib.lean,Mathlib/CategoryTheory/LocallyCartesianClosed/Basic.lean,Mathlib/CategoryTheory/LocallyCartesianClosed/ChosenPullbacksAlong.lean,Mathlib/CategoryTheory/LocallyCartesianClosed/ExponentiableMorphism.lean,Mathlib/CategoryTheory/LocallyCartesianClosed/Sections.lean 5 9 ['Jlh18', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'sinhp'] nobody
9-59712
9 days ago
unknown
unknown
32991 artie2000
author:artie2000
chore(Algebra/Algebra): remove `Algebra.cast` coercion See discussion at https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Algebra.2Ecast/with/564501144 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict
label:t-algebra$
32/125 Mathlib/Algebra/Algebra/Basic.lean,Mathlib/Algebra/Algebra/Defs.lean,Mathlib/Algebra/Algebra/Field.lean,Mathlib/Algebra/Algebra/Subalgebra/Lattice.lean,Mathlib/Algebra/BigOperators/Expect.lean,Mathlib/Analysis/Normed/Algebra/Ultra.lean,Mathlib/FieldTheory/Differential/Liouville.lean,Mathlib/LinearAlgebra/Ray.lean,Mathlib/RingTheory/Localization/FractionRing.lean 9 11 ['Vierkantor', 'artie2000', 'github-actions', 'mathlib4-merge-conflict-bot', 'plp127', 'vihdzp'] Vierkantor
assignee:Vierkantor
9-58766
9 days ago
unknown
unknown
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 WIP t-number-theory t-algebra merge-conflict
label:t-algebra$
188/87 Mathlib/NumberTheory/NumberField/FinitePlaces.lean,Mathlib/NumberTheory/Padics/WithVal.lean,Mathlib/RingTheory/DedekindDomain/AdicValuation.lean,Mathlib/RingTheory/DedekindDomain/FiniteAdeleRing.lean,Mathlib/RingTheory/LaurentSeries.lean,Mathlib/Topology/Algebra/Valued/WithVal.lean 6 8 ['github-actions', 'leanprover-bot', 'mathlib4-merge-conflict-bot', 'smmercuri'] nobody
9-57459
9 days ago
119-79169
119 days ago
3-78107
3 days
32585 CBirkbeck
author:CBirkbeck
feat(NumberTheory/ModularForms/EisensteinSeries/E2/Transform): E2 under the action of SL2 We show how E2 transforms under the slash action of SL2. --- - [x] depends on : #32584 - [x] depends on : #32955 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 466/0 Mathlib.lean,Mathlib/NumberTheory/ModularForms/EisensteinSeries/E2/Summable.lean,Mathlib/NumberTheory/ModularForms/EisensteinSeries/E2/Transform.lean 3 11 ['CBirkbeck', 'github-actions', 'loefflerd', 'mathlib4-merge-conflict-bot'] loefflerd
assignee:loefflerd
9-56315
9 days ago
9-56315
9 days ago
12-53590
12 days
33490 YaelDillies
author:YaelDillies
refactor(Data/Finsupp): remove `DecidableEq` argument from `curry` This is motivated by it spuriously requiring extra decidability assumptions in group cohomology. This partially reverts #24746. No motivation was given there for why computability was necessary. `Finsupp.curry` will be made computable again anyway once `Finsupp` is redefined to be `DFinsupp`. From ClassFieldTheory --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) CFT t-data 15/21 Mathlib/Data/Finsupp/Basic.lean,Mathlib/LinearAlgebra/Finsupp/Defs.lean,Mathlib/LinearAlgebra/Finsupp/LinearCombination.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/Basic.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/FiniteCyclic.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/Shapiro.lean,Mathlib/RepresentationTheory/Homological/Resolution.lean,Mathlib/RepresentationTheory/Rep.lean,Mathlib/RingTheory/AlgebraTower.lean 9 5 ['YaelDillies', 'eric-wieser', 'github-actions', 'tb65536'] nobody
9-50007
9 days ago
11-79369
11 days ago
11-79189
11 days
17176 arulandu
author:arulandu
feat: integrals and integrability with .re Lemmas for swapping order of .re and integration/integrability. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author new-contributor t-measure-probability please-adopt 49/0 Mathlib/MeasureTheory/Function/L1Space.lean,Mathlib/MeasureTheory/Integral/IntegrableOn.lean,Mathlib/MeasureTheory/Integral/IntervalIntegral.lean,Mathlib/MeasureTheory/Integral/SetIntegral.lean 4 32 ['EtienneC30', 'arulandu', 'github-actions', 'loefflerd'] nobody
9-49291
9 days ago
unknown
unknown
32918 michelsol
author:michelsol
feat: define `supEdist` and `supDist` Create a new file Topology.MetricSpace.SupDistance and define the supremal distance in (extended) metric spaces. The defined `supEdist` and `supDist` will have similar theory to the already existing `infEdist` and `infDist`. The motivation is to be able to define the radius of a minimal bounding sphere as the infimum of the supDist later. [zulip discussion here](https://leanprover.zulipchat.com/#narrow/channel/116395-maths/topic/Formalizing.20Jung's.20theorem.20and.20minimal.20bounding.20spheres) t-topology new-contributor merge-conflict 75/0 Mathlib.lean,Mathlib/Topology/MetricSpace/SupDistance.lean 2 2 ['github-actions', 'mathlib4-merge-conflict-bot'] RemyDegenne
assignee:RemyDegenne
9-48692
9 days ago
9-48694
9 days ago
21-957
21 days
33100 themathqueen
author:themathqueen
refactor(Algebra/Order/Field/Basic): generalize file from `LinearOrder` to `PartialOrder` and `PosMulReflectLT` It's a well-known easy fact that there is no way to equip `ℂ` with a *linear* order satisfying `IsStrictOrderedRing`. However, it is equipped with a partial order (available in the `ComplexOrder` namespace) given by `a ≤ b ↔ a.re ≤ b.re ∧ a.im = b.im`. This order satisfies `IsStrictOrderedRing`. However, it has some other nice properties, for instance `0 < a⁻¹ ↔ 0 < a` (because it is a `GroupWithZero` satisfying `PosMulReflectLT` so `inv_pos` applies), and moreover, in this PR we also show that a (partially) ordered field with this property satisfies `a⁻¹ < 0 ↔ a < 0`. This means that the field operation is well-behaved in regards to elements comparable with zero. This PR refactors `Algebra/Order/Field/Basic.lean` so that it applies to *partially* ordered fields that in addition satisfy `PosMulReflectLT` (e.g., `ℂ`). The vast majority of the lemmas are applicable in this more general setting, albeit with refactored proofs. The diff is a bit messy, but it's easy to understand with the right point-of-view: 1. lemmas which require linear orders are grouped into their own sections below the corresponding sections for partially ordered fields 2. proofs are refactored with the weaker hypotheses 3. a few lemmas near the top didn't actually need `IsStrictOrderedRing`, so those are grouped at the top. 4. The only new declarations added are `inv_lt_zero'` and `inv_nonpos'`, no others were deleted or changed (aside from weakening type class assumptions). 5. The positivity extension at the bottom of the file has its type class requirements weakened so that it applies in more contexts. Co-authored-by: Jireh Loreaux --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
180/131 Mathlib/Algebra/Order/Field/Basic.lean 1 6 ['github-actions', 'j-loreaux', 'leanprover-radar', 'mathlib4-merge-conflict-bot', 'themathqueen'] dagurtomas
assignee:dagurtomas
9-48187
9 days ago
9-45330
9 days ago
26-37131
26 days
33586 CoolRmal
author:CoolRmal
feat: Lower Limit Topology --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology 328/0 Mathlib.lean,Mathlib/Topology/Order/LowerUpperLimitTopology.lean 2 10 ['CoolRmal', 'github-actions', 'plp127'] nobody
9-47993
9 days ago
unknown
unknown
33608 riccardobrasca
author:riccardobrasca
feat: generalize universes in representation theory (#33598) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-algebra
label:t-algebra$
53/52 Mathlib/Algebra/Category/ModuleCat/Adjunctions.lean,Mathlib/RepresentationTheory/Coinduced.lean,Mathlib/RepresentationTheory/FinGroupCharZero.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/Basic.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/Shapiro.lean,Mathlib/RepresentationTheory/Homological/GroupHomology/Basic.lean,Mathlib/RepresentationTheory/Homological/GroupHomology/LowDegree.lean,Mathlib/RepresentationTheory/Induced.lean,Mathlib/RepresentationTheory/Invariants.lean,Mathlib/RepresentationTheory/Rep.lean 10 4 ['github-actions', 'leanprover-radar', 'riccardobrasca'] nobody
9-44959
9 days ago
unknown
unknown
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 - [x] depends on: #29230 for `Lattice` `CompleteLattice` - [ ] depends on: #29241 for the definition of `orthogonal` blocked-by-other-PR 243/6 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
9-43980
9 days ago
134-72213
134 days ago
0-1521
25 minutes
33619 vihdzp
author:vihdzp
refactor: flip `Ixx_def` theorems This sort of `_def` theorems are generally written so that the defined constant is on the LHS. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order awaiting-CI 11/13 Mathlib/Algebra/Module/Submodule/Pointwise.lean,Mathlib/Order/Interval/Set/Defs.lean,Mathlib/Topology/Path.lean 3 1 ['github-actions'] nobody
9-42297
9 days ago
unknown
unknown
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. blocked-by-other-PR t-measure-probability 668/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
9-40145
9 days ago
unknown
unknown
33010 xgenereux
author:xgenereux
feat: localizations of primes in Dedekind domains are valuation subrings The goal of this PR is the theorem `valuationSubringAtPrime_eq_valuationSubring` which states that the localization at a nonzero prime in a Dedekind domain is precisely the valuation subring of the valuation associated with that same prime. Given a Dedekind domain `R` in its field of fractions `K`, we define `IsDedekindDomain.valuationSubringAtPrime`, which is the localization of `R` at a nonzero prime, viewed as valuation subring of `K`. We show that `valuationSubringAtPrime K v ≤ (valuation K v).valuationSubring` and use maximality to show that they must be equal. Other small note: - added a variant of `intValuation_exists_uniformizer` in terms of `valuation` (instead of intValuation). Co-authored-by: María Inés de Frutos Fernández <[mariaines.dff@gmail.com](mailto:mariaines.dff@gmail.com)> --- - [ ] depends on: #33634 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-ring-theory large-import awaiting-author WIP blocked-by-other-PR 96/4 Mathlib/RingTheory/DedekindDomain/AdicValuation.lean 1 9 ['erdOne', 'github-actions', 'mathlib4-dependent-issues-bot', 'xgenereux'] nobody
9-39121
9 days ago
26-24718
26 days ago
2-22032
2 days
33557 ocfnash
author:ocfnash
feat: existence of bases for root pairings --- Currently terrible mess. Will return to tidy up in due course. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-algebra
label:t-algebra$
334/85 Mathlib/Algebra/Group/Irreducible/Indecomposable.lean,Mathlib/LinearAlgebra/RootSystem/BaseExists.lean,Mathlib/LinearAlgebra/RootSystem/Finite/Nondegenerate.lean 3 1 ['github-actions'] nobody
9-37948
9 days ago
unknown
unknown
33281 michelsol
author:michelsol
feat(Analysis/SpecialFunctions/Integrals): integral of 1/sqrt(1-x^2) and its integrability. Add the integral of the derivative of arcsin and its integrability. --- - [ ] depends on: #33280 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor blocked-by-other-PR merge-conflict 59/0 Mathlib/Analysis/SpecialFunctions/Integrability/Basic.lean,Mathlib/Analysis/SpecialFunctions/Integrals/Basic.lean,Mathlib/MeasureTheory/Integral/IntervalIntegral/FundThmCalculus.lean 3 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
9-35221
9 days ago
20-54035
20 days ago
0-811
13 minutes
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-data
label:t-algebra$
119/60 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 9 12 ['alreadydone', 'astrainfinita', 'github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'mathlib4-merge-conflict-bot'] pechersky
assignee:pechersky
9-33695
9 days ago
9-30861
9 days ago
44-3483
44 days
33252 SnirBroshi
author:SnirBroshi
feat(Combinatorics/SimpleGraph/Clique): cliques & independent sets are chains & antichains --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics 11/0 Mathlib/Combinatorics/SimpleGraph/Clique.lean,Mathlib/Combinatorics/SimpleGraph/Coloring.lean 2 1 ['github-actions'] nobody
9-32318
9 days ago
unknown
unknown
33458 NoneMore
author:NoneMore
feat(ModelTheory): add lifting for embeddings to languages with constants Prepare for a generalized Tarski-Vaught test with a set as input instead of a substructure. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-logic new-contributor 46/0 Mathlib/ModelTheory/ElementaryMaps.lean,Mathlib/ModelTheory/LanguageMap.lean 2 1 ['github-actions'] fpvandoorn
assignee:fpvandoorn
9-31254
9 days ago
13-1906
13 days ago
13-1726
13 days
33487 gasparattila
author:gasparattila
feat(Topology/UniformSpace): `SetRel.{inv,image,preimage}` of `entourageProd` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology 15/0 Mathlib/Topology/UniformSpace/Basic.lean 1 1 ['github-actions'] dagurtomas
assignee:dagurtomas
9-31249
9 days ago
12-61980
12 days ago
12-61800
12 days
33494 vihdzp
author:vihdzp
feat(RingTheory/HahnSeries/Basic): more theorems on `order`/`orderTop` We also deprecate various badly named or overspecific theorems relating to `ofSuppBddBelow`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-ring-theory 64/32 Mathlib/Algebra/Vertex/VertexOperator.lean,Mathlib/RingTheory/HahnSeries/Basic.lean,Mathlib/RingTheory/LaurentSeries.lean 3 1 ['github-actions'] mattrobball
assignee:mattrobball
9-31248
9 days ago
10-310
10 days ago
10-130
10 days
24129 urkud
author:urkud
feat: symmetry of Gateaux derivatives --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis 189/1 Mathlib/Analysis/Calculus/LineDeriv/Basic.lean,Mathlib/Analysis/Calculus/LineDeriv/Symmetric.lean 2 2 ['github-actions', 'mathlib4-merge-conflict-bot'] nobody
9-24843
9 days ago
unknown
unknown
33644 vihdzp
author:vihdzp
feat(Analysis/Real/Hyperreal): more lemmas on `Tendsto` I've taken care to neither state or prove these using the various specialized predicates for `Hyperreal`, such as `Infinitesimal`, `Infinite`, `IsSt`. These will be deprecated in a followup PR in favor of reasoning with `ArchimedeanClass.mk` and `ArchimedeanClass.stdPart`. --- - [ ] depends on: #33649 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis large-import blocked-by-other-PR 199/30 Mathlib/Algebra/Order/AddGroupWithTop.lean,Mathlib/Algebra/Order/Ring/Archimedean.lean,Mathlib/Algebra/Order/Ring/StandardPart.lean,Mathlib/Analysis/Real/Hyperreal.lean 4 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
9-16581
9 days ago
9-22870
9 days ago
0-3677
1 hour
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-ring-theory awaiting-author 105/0 Mathlib.lean,Mathlib/RingTheory/Flat/IsBaseChange.lean 2 9 ['Thmoas-Guan', 'erdOne', 'github-actions', 'mathlib4-merge-conflict-bot', 'urkud'] nobody
9-10774
9 days ago
53-37038
53 days ago
16-38821
16 days
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR large-import 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
9-10681
9 days ago
unknown
unknown
33650 vihdzp
author:vihdzp
refactor: deprecate bespoke `Hyperreal` machinery Currently, these six definitions are in the `Hyperreal` namespace: - `IsSt x r`: a predicate for `r` being a standard part of `x` - `st x`: the standard part of `x` - `Infinitesimal x`: predicate for infinitesimal elements - `InfinitePos x`: predicate for infinite and positive elements - `InfiniteNeg x`: predicate for infinite and negative elements - `Infinite x`: predicate for infinite (positive or negative) elements. We deprecate all six of these and all of their API, in favor of reasoning with [`ArchimedeanClass`](https://leanprover-community.github.io/mathlib4_docs/Mathlib/Algebra/Order/Archimedean/Class.html#ArchimedeanClass) and [`ArchimedeanClass.stdPart`](https://leanprover-community.github.io/mathlib4_docs/Mathlib/Algebra/Order/Ring/StandardPart.html#ArchimedeanClass.stdPart). The replacements are as follows: - `IsSt x r`: `0 ≤ ArchimedeanClass.mk x ∧ stdPart x = r` - `st x`: `stdPart x` - `Infinitesimal x`: `0 < ArchimedeanClass.mk x` - `InfinitePos x`: `0 < x ∧ ArchimedeanClass.mk x < 0` - `InfiniteNeg x`: `x < 0 ∧ ArchimedeanClass.mk x < 0` - `Infinite x`: `ArchimedeanClass.mk x < 0` All of these equivalences are proved within the PR, though these new theorems have also been insta-deprecated. Most of the existing API on these predicates was largely uninteresting boilerplate, and has been deprecated without replacement. For the few results of mathematical interest (those whose proofs are longer than a few lines), I've golfed their proofs as a stress test to ensure that this new API is capable of easily proving them. --- - [ ] depends on: #33644 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra large-import blocked-by-other-PR
label:t-algebra$
1053/579 Mathlib.lean,Mathlib/Algebra/Order/AddGroupWithTop.lean,Mathlib/Algebra/Order/Ring/Archimedean.lean,Mathlib/Algebra/Order/Ring/StandardPart.lean,Mathlib/Analysis/Real/Hyperreal.lean,Mathlib/Deprecated/Hyperreal.lean 6 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
9-7592
9 days ago
unknown
unknown
26214 Thmoas-Guan
author:Thmoas-Guan
feat(Algebra): definition of depth In this PR, we defined the depth of two modules as the minimal order of nonvanishing `Ext` and the `I-depth` for ideal `I` and some basic properties. Including the equivalence of the two in the condition of rees theorem. --- - [ ] depends on: #26212 - [ ] depends on: #32966 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra blocked-by-other-PR large-import
label:t-algebra$
610/16 Mathlib/RingTheory/Regular/Category.lean,Mathlib/RingTheory/Regular/Depth.lean 2 7 ['Thmoas-Guan', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
9-5425
9 days 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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra blocked-by-other-PR large-import
label:t-algebra$
894/16 Mathlib/RingTheory/Regular/Category.lean,Mathlib/RingTheory/Regular/Depth.lean 2 7 ['Thmoas-Guan', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
9-5290
9 days ago
unknown
unknown
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. --- - [x] depends on: #31998 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 243/0 Mathlib.lean,Mathlib/RingTheory/LocalProperties/ProjectiveDimension.lean 2 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
9-3082
9 days ago
9-11219
9 days ago
13-18336
13 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 - [x] depends on: #31696 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra blocked-by-other-PR t-category-theory
label:t-algebra$
341/0 Mathlib.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/Pretriangulated.lean,Mathlib/Algebra/Homology/HomotopyCategory/ShortExact.lean 6 5 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
9-1736
9 days ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra blocked-by-other-PR t-category-theory
label:t-algebra$
640/0 Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Ext/Ulift.lean,Mathlib/Algebra/Category/ModuleCat/Ulift.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/Pretriangulated.lean,Mathlib/Algebra/Homology/HomotopyCategory/ShortExact.lean 8 5 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
9-1587
9 days ago
unknown
unknown
33061 edwin1729
author:edwin1729
refactor: generalise compact from CompleteLattice to PartialOrder `IsCompactElement` assumes a `CompleteLattice` structure on the type for which it is defined. But a `PartialOrder` will suffice and this is the textbook definition of compact https://en.wikipedia.org/wiki/Compact_element. Also it is currently defined in a non-standard way. The standard definition uses directed sets. Changing this has indeed simplified most proofs by removing an `rw` into this more standard form. --- Note to reviewers: moving `IsCompactElement` out of the `CompleteLattice` namespace caused the loss of being able to use dot notation [here](https://github.com/leanprover-community/mathlib4/pull/33061/changes#diff-2e06453359871b8a74315294d1f7825b7b5aa1221c69b4e058893b2c9418230fR498) and [here](https://github.com/leanprover-community/mathlib4/pull/33061/changes#diff-1d4a166e29849096ebe0e5d25bd4dc5f97db1d3b8caf1703177034160e77a310R350). Would like help fixing that [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor awaiting-author 84/63 Mathlib/Algebra/Lie/Submodule.lean,Mathlib/LinearAlgebra/Span/Basic.lean,Mathlib/Order/BooleanGenerators.lean,Mathlib/Order/CompactlyGenerated/Basic.lean,Mathlib/Order/CompactlyGenerated/Intervals.lean,Mathlib/RingTheory/Finiteness/Basic.lean,Mathlib/RingTheory/Ideal/Span.lean,Mathlib/RingTheory/Spectrum/Prime/Topology.lean,Mathlib/Topology/Sets/Opens.lean 9 11 ['b-mehta', 'edwin1729', 'github-actions', 'plp127'] nobody
8-84556
8 days ago
26-61186
26 days ago
0-70180
19 hours
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra blocked-by-other-PR t-category-theory
label:t-algebra$
170/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,Mathlib/Algebra/Homology/ShortComplex/ModuleCat.lean,Mathlib/RingTheory/Noetherian/Basic.lean 7 9 ['Thmoas-Guan', 'dagurtomas', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
8-79435
8 days ago
unknown
unknown
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. --- - [ ] depends on: #32316 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra blocked-by-other-PR
label:t-algebra$
254/0 Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Ext/DimensionShifting.lean,Mathlib/Algebra/Category/ModuleCat/ProjectiveDimension.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/EnoughInjectives.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/EnoughProjectives.lean,Mathlib/Algebra/Homology/ShortComplex/ModuleCat.lean,Mathlib/RingTheory/Noetherian/Basic.lean 7 7 ['Thmoas-Guan', 'dagurtomas', 'github-actions', 'mathlib4-dependent-issues-bot'] dagurtomas
assignee:dagurtomas
8-79397
8 days ago
49-48307
49 days ago
5-40614
5 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. --- - [ ] depends on: #32316 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-category-theory awaiting-author blocked-by-other-PR
label:t-algebra$
264/0 Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Baer.lean,Mathlib/Algebra/Category/ModuleCat/Ext/DimensionShifting.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/EnoughInjectives.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/EnoughProjectives.lean,Mathlib/Algebra/Homology/ShortComplex/ModuleCat.lean,Mathlib/RingTheory/Noetherian/Basic.lean 7 4 ['github-actions', 'joelriou', 'mathlib4-dependent-issues-bot'] dagurtomas
assignee:dagurtomas
8-79318
8 days ago
44-51139
44 days ago
7-12721
7 days
33640 JovanGerb
author:JovanGerb
feat: tool for finding duplicate declarations This PR defines a tool for finding duplicate declarations automatically. This can be used to help fix this technical debt. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta 176/0 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/DuplicateDecls.lean 3 1 ['github-actions'] nobody
8-78769
8 days ago
unknown
unknown
26215 Thmoas-Guan
author:Thmoas-Guan
feat(Algebra): Auslander–Buchsbaum theorem This PR mainly proved the Auslander-Buchsbaum theorem stating for a noetherian local ring `R` and a finitely generated `R` module `M` , `proj.dim(M) + depth(M) = depth(R)`. Co-authored-by: Yongle Hu --- - [ ] depends on: #26214 - [ ] depends on: #32316 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra blocked-by-other-PR large-import
label:t-algebra$
1166/16 Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Ext/DimensionShifting.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/EnoughInjectives.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/EnoughProjectives.lean,Mathlib/Algebra/Homology/ShortComplex/ModuleCat.lean,Mathlib/RingTheory/Noetherian/Basic.lean,Mathlib/RingTheory/Regular/AuslanderBuchsbaum.lean,Mathlib/RingTheory/Regular/Category.lean,Mathlib/RingTheory/Regular/Depth.lean 9 8 ['Thmoas-Guan', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
8-78719
8 days ago
unknown
unknown
26217 Thmoas-Guan
author:Thmoas-Guan
feat(Algebra): Ischebeck theorem This PR mainly proved the Ischbecke theorem, stating that `depth(N,M)` is greater or equal to `depth(M) - dim(N)` for finitely generated module `N, M` over local ring. --- - [ ] depends on: #26214 - [ ] depends on: #32081 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra blocked-by-other-PR large-import
label:t-algebra$
1056/16 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/Algebra/Homology/ShortComplex/ModuleCat.lean,Mathlib/RingTheory/Noetherian/Basic.lean,Mathlib/RingTheory/Regular/Category.lean,Mathlib/RingTheory/Regular/Depth.lean,Mathlib/RingTheory/Regular/Ischebeck.lean 10 8 ['Thmoas-Guan', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
8-78350
8 days ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import awaiting-author t-ring-theory 220/16 Mathlib/RingTheory/Regular/Category.lean,Mathlib/RingTheory/Regular/Depth.lean 2 41 ['Thmoas-Guan', 'alreadydone', 'dagurtomas', 'erdOne', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
8-78336
8 days ago
11-46682
11 days ago
58-41156
58 days
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra blocked-by-other-PR large-import
label:t-algebra$
1980/26 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/Algebra/Homology/ShortComplex/ModuleCat.lean,Mathlib/Algebra/Order/Monoid/Unbundled/WithTop.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/RingTheory/CohenMacaulay/Basic.lean,Mathlib/RingTheory/Noetherian/Basic.lean,Mathlib/RingTheory/Regular/Category.lean,Mathlib/RingTheory/Regular/Depth.lean,Mathlib/RingTheory/Regular/Ischebeck.lean 13 14 ['Thmoas-Guan', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
8-78322
8 days ago
unknown
unknown
28599 Thmoas-Guan
author:Thmoas-Guan
feat(RingTheory): polynomial over CM ring is CM polynomial over Cohen Macaulay ring is Cohen Macaulay --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-ring-theory large-import 2197/26 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/Algebra/Homology/ShortComplex/ModuleCat.lean,Mathlib/Algebra/Order/Monoid/Unbundled/WithTop.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/RingTheory/CohenMacaulay/Basic.lean,Mathlib/RingTheory/CohenMacaulay/Polynomial.lean,Mathlib/RingTheory/Noetherian/Basic.lean,Mathlib/RingTheory/Regular/Category.lean,Mathlib/RingTheory/Regular/Depth.lean,Mathlib/RingTheory/Regular/Ischebeck.lean 14 9 ['github-actions', 'mathlib4-merge-conflict-bot'] nobody
8-78228
8 days ago
unknown
unknown
26245 Thmoas-Guan
author:Thmoas-Guan
feat(Algebra): cohen macaulay local ring is catenary We prove Cohen Macaulay local ring is catenary. Following Theorem 31, Chater 6, _Commutative Algebra_, Matsumura --- - [ ] depends on: #26218 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-algebra blocked-by-other-PR large-import
label:t-algebra$
2375/26 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/Algebra/Homology/ShortComplex/ModuleCat.lean,Mathlib/Algebra/Order/Monoid/Unbundled/WithTop.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/RingTheory/CohenMacaulay/Basic.lean,Mathlib/RingTheory/CohenMacaulay/Catenary.lean,Mathlib/RingTheory/Noetherian/Basic.lean,Mathlib/RingTheory/Regular/Category.lean,Mathlib/RingTheory/Regular/Depth.lean,Mathlib/RingTheory/Regular/Ischebeck.lean 14 14 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
8-78209
8 days ago
unknown
unknown
26957 Thmoas-Guan
author:Thmoas-Guan
feat(Algebra): unmixed thm of Cohen-Macaulay ring In this PR we proved for a (comm)ring `R`, `R` is Cohen-Macaulay ring iff the unmixed theorem holds (for every ideal `I` of height `r` generated by `r` elements, all associated primes of `R/I` have height `r` ) --- - [ ] depends on: #26245 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra blocked-by-other-PR large-import
label:t-algebra$
2556/26 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/Algebra/Homology/ShortComplex/ModuleCat.lean,Mathlib/Algebra/Order/Monoid/Unbundled/WithTop.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/RingTheory/CohenMacaulay/Basic.lean,Mathlib/RingTheory/CohenMacaulay/Catenary.lean,Mathlib/RingTheory/CohenMacaulay/Unmixed.lean,Mathlib/RingTheory/Noetherian/Basic.lean,Mathlib/RingTheory/Regular/Category.lean,Mathlib/RingTheory/Regular/Depth.lean,Mathlib/RingTheory/Regular/Ischebeck.lean 15 12 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
8-78197
8 days ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra blocked-by-other-PR
label:t-algebra$
1012/0 Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Baer.lean,Mathlib/Algebra/Category/ModuleCat/Ext/DimensionShifting.lean,Mathlib/Algebra/Category/ModuleCat/Ext/Ulift.lean,Mathlib/Algebra/Category/ModuleCat/InjectiveDimension.lean,Mathlib/Algebra/Category/ModuleCat/Ulift.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/Bijection.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/EnoughInjectives.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/EnoughProjectives.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/Map.lean,Mathlib/Algebra/Homology/DerivedCategory/ShortExact.lean,Mathlib/Algebra/Homology/HomotopyCategory/Pretriangulated.lean,Mathlib/Algebra/Homology/HomotopyCategory/ShortExact.lean,Mathlib/Algebra/Homology/ShortComplex/ModuleCat.lean,Mathlib/RingTheory/Noetherian/Basic.lean 15 4 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
8-76536
8 days 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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-ring-theory blocked-by-other-PR 480/10 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/Algebra/Homology/ShortComplex/ModuleCat.lean,Mathlib/Algebra/Order/Monoid/Unbundled/WithTop.lean,Mathlib/CategoryTheory/Abelian/Projective/Dimension.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/RingTheory/Noetherian/Basic.lean,Mathlib/RingTheory/Regular/ProjectiveDimension.lean 11 27 ['Thmoas-Guan', 'erdOne', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
8-76412
8 days ago
60-60014
60 days ago
0-20294
5 hours
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR 1108/10 Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Baer.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/Algebra/Homology/DerivedCategory/Ext/Map.lean,Mathlib/Algebra/Homology/DerivedCategory/ShortExact.lean,Mathlib/Algebra/Homology/HomotopyCategory/Pretriangulated.lean,Mathlib/Algebra/Homology/HomotopyCategory/ShortExact.lean,Mathlib/Algebra/Homology/ShortComplex/ModuleCat.lean,Mathlib/Algebra/Order/Monoid/Unbundled/WithTop.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/RingTheory/Noetherian/Basic.lean,Mathlib/RingTheory/Regular/InjectiveDimension.lean 15 4 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
8-74751
8 days ago
50-71451
50 days ago
0-294
4 minutes
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR 1099/0 Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Baer.lean,Mathlib/Algebra/Category/ModuleCat/Ext/DimensionShifting.lean,Mathlib/Algebra/Category/ModuleCat/Ext/Ulift.lean,Mathlib/Algebra/Category/ModuleCat/InjectiveDimension.lean,Mathlib/Algebra/Category/ModuleCat/Ulift.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/Bijection.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/EnoughInjectives.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/EnoughProjectives.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/Map.lean,Mathlib/Algebra/Homology/DerivedCategory/ShortExact.lean,Mathlib/Algebra/Homology/HomotopyCategory/Pretriangulated.lean,Mathlib/Algebra/Homology/HomotopyCategory/ShortExact.lean,Mathlib/Algebra/Homology/ShortComplex/ModuleCat.lean,Mathlib/RingTheory/Gorenstein/Defs.lean,Mathlib/RingTheory/Noetherian/Basic.lean 16 4 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
8-74388
8 days ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-ring-theory awaiting-author 231/0 Mathlib.lean,Mathlib/RingTheory/LocalProperties/Injective.lean 2 9 ['Thmoas-Guan', 'dagurtomas', 'erdOne', 'github-actions'] erdOne
assignee:erdOne
8-74299
8 days ago
11-61085
11 days ago
8-56552
8 days
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR 450/0 Mathlib.lean,Mathlib/RingTheory/LocalProperties/Injective.lean,Mathlib/RingTheory/LocalProperties/InjectiveDimension.lean 3 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
8-74230
8 days ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR 1651/0 Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Baer.lean,Mathlib/Algebra/Category/ModuleCat/Ext/DimensionShifting.lean,Mathlib/Algebra/Category/ModuleCat/Ext/Ulift.lean,Mathlib/Algebra/Category/ModuleCat/InjectiveDimension.lean,Mathlib/Algebra/Category/ModuleCat/Ulift.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/Bijection.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/EnoughInjectives.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/EnoughProjectives.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/Map.lean,Mathlib/Algebra/Homology/DerivedCategory/ShortExact.lean,Mathlib/Algebra/Homology/HomotopyCategory/Pretriangulated.lean,Mathlib/Algebra/Homology/HomotopyCategory/ShortExact.lean,Mathlib/Algebra/Homology/ShortComplex/ModuleCat.lean,Mathlib/RingTheory/Gorenstein/Basic.lean,Mathlib/RingTheory/Gorenstein/Defs.lean,Mathlib/RingTheory/LocalProperties/Injective.lean,Mathlib/RingTheory/LocalProperties/InjectiveDimension.lean,Mathlib/RingTheory/Noetherian/Basic.lean 19 5 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
8-74159
8 days ago
unknown
unknown
32959 CBirkbeck
author:CBirkbeck
feat(NumberTheory/ModularForms/QExpansion): define qExpansion ring hom and some more API We construct the ring homomorphism from the graded ring of modular forms to power series. We prove develop some basic API for this and also prove the qExpansion coefficients are unique, which is useful to extracting the actual qExpansions of Eisenstein series. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-number-theory 410/6 Mathlib/Analysis/Calculus/Deriv/Mul.lean,Mathlib/Analysis/Calculus/IteratedDeriv/Lemmas.lean,Mathlib/NumberTheory/ModularForms/QExpansion.lean 3 1 ['github-actions'] loefflerd
assignee:loefflerd
8-72768
8 days ago
8-71903
8 days ago
15-2192
15 days
33369 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`. --- - [ ] depends on: #31046 - [ ] depends on: #31222 - [ ] depends on: #32316 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import blocked-by-other-PR 948/0 Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Ext/BaseChange.lean,Mathlib/Algebra/Category/ModuleCat/Ext/DimensionShifting.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/EnoughInjectives.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/EnoughProjectives.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/Map.lean,Mathlib/Algebra/Homology/DerivedCategory/ShortExact.lean,Mathlib/Algebra/Homology/HomotopyCategory/Pretriangulated.lean,Mathlib/Algebra/Homology/HomotopyCategory/ShortExact.lean,Mathlib/Algebra/Homology/ShortComplex/ModuleCat.lean,Mathlib/Algebra/Module/FinitePresentation.lean,Mathlib/RingTheory/Flat/IsBaseChange.lean,Mathlib/RingTheory/Noetherian/Basic.lean 13 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
8-72081
8 days ago
16-77822
16 days ago
0-535
8 minutes
33377 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: #33369 - [ ] depends on: #31884 - [ ] depends on: #32098 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import blocked-by-other-PR 2590/10 Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Baer.lean,Mathlib/Algebra/Category/ModuleCat/Ext/BaseChange.lean,Mathlib/Algebra/Category/ModuleCat/Ext/DimensionShifting.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/Ext/Bijection.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/EnoughInjectives.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/EnoughProjectives.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/Map.lean,Mathlib/Algebra/Homology/DerivedCategory/ShortExact.lean,Mathlib/Algebra/Homology/HomotopyCategory/Pretriangulated.lean,Mathlib/Algebra/Homology/HomotopyCategory/ShortExact.lean,Mathlib/Algebra/Homology/ShortComplex/ModuleCat.lean,Mathlib/Algebra/Module/FinitePresentation.lean,Mathlib/Algebra/Order/Monoid/Unbundled/WithTop.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/RingTheory/Flat/IsBaseChange.lean,Mathlib/RingTheory/Gorenstein/Defs.lean,Mathlib/RingTheory/Gorenstein/Polynomial.lean,Mathlib/RingTheory/Noetherian/Basic.lean,Mathlib/RingTheory/Regular/InjectiveDimension.lean 24 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
8-71895
8 days ago
unknown
unknown
33379 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: #31884 - [ ] depends on: #26218 - [ ] depends on: #32098 - [ ] depends on: #31644 - [ ] depends on: #33369 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import blocked-by-other-PR 5059/26 Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Baer.lean,Mathlib/Algebra/Category/ModuleCat/Ext/BaseChange.lean,Mathlib/Algebra/Category/ModuleCat/Ext/DimensionShifting.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/Ext/Bijection.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/EnoughInjectives.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/EnoughProjectives.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/Map.lean,Mathlib/Algebra/Homology/DerivedCategory/ShortExact.lean,Mathlib/Algebra/Homology/HomotopyCategory/Pretriangulated.lean,Mathlib/Algebra/Homology/HomotopyCategory/ShortExact.lean,Mathlib/Algebra/Homology/ShortComplex/ModuleCat.lean,Mathlib/Algebra/Module/FinitePresentation.lean,Mathlib/Algebra/Order/Monoid/Unbundled/WithTop.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/Noetherian/Basic.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 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
8-71760
8 days ago
unknown
unknown
33380 Thmoas-Guan
author:Thmoas-Guan
feat(RingTheory): Gorenstein local ring is Cohen--Macaulay local ring of type one 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: #33379 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import blocked-by-other-PR 6010/26 Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Baer.lean,Mathlib/Algebra/Category/ModuleCat/Ext/BaseChange.lean,Mathlib/Algebra/Category/ModuleCat/Ext/DimensionShifting.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/Ext/Bijection.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/EnoughInjectives.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/EnoughProjectives.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/Map.lean,Mathlib/Algebra/Homology/DerivedCategory/ShortExact.lean,Mathlib/Algebra/Homology/HomotopyCategory/Pretriangulated.lean,Mathlib/Algebra/Homology/HomotopyCategory/ShortExact.lean,Mathlib/Algebra/Homology/ShortComplex/ModuleCat.lean,Mathlib/Algebra/Module/FinitePresentation.lean,Mathlib/Algebra/Order/Monoid/Unbundled/WithTop.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/Noetherian/Basic.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 31 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
8-71653
8 days ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-ring-theory blocked-by-other-PR 164/0 Mathlib.lean,Mathlib/RingTheory/Ideal/Cotangent.lean,Mathlib/RingTheory/RegularLocalRing/Defs.lean,Mathlib/RingTheory/RegularLocalRing/RegularRing/Basic.lean 4 5 ['Thmoas-Guan', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
8-71360
8 days 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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-ring-theory blocked-by-other-PR 512/14 Mathlib.lean,Mathlib/Algebra/Order/Monoid/Unbundled/WithTop.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/RingTheory/Ideal/Cotangent.lean,Mathlib/RingTheory/KrullDimension/Regular.lean,Mathlib/RingTheory/RegularLocalRing/Basic.lean,Mathlib/RingTheory/RegularLocalRing/Defs.lean 7 5 ['Thmoas-Guan', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
8-71297
8 days 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` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data awaiting-author 58/10 Mathlib/Algebra/Order/Monoid/Unbundled/WithTop.lean,Mathlib/Data/ENat/Basic.lean 2 27 ['Ruben-VandeVelde', 'Thmoas-Guan', 'YaelDillies', 'alreadydone', 'erdOne', 'github-actions', 'pechersky', 'urkud'] pechersky
assignee:pechersky
8-70920
8 days ago
8-70920
8 days ago
56-34514
56 days
33257 NickAdfor
author:NickAdfor
feat(Combinatorics/SimpleGraph/Bipartite): Odd Cycle Theorem (A Solution to TODO) Prove bipartite iff all cycles are even This PR formalizes the classical graph theory theorem: a graph is bipartite if and only if all its cycles have even length. Co-authored-by: Nick Adfor Co-authored-by: Yue Sun Co-authored-by: Aristotle AI --- ## Main results - `SimpleGraph.bipartite_iff_all_cycles_even` : the main equivalence theorem ## Key supporting lemmas - `SimpleGraph.even_length_iff_same_color` : parity lemma for 2-colorings - `SimpleGraph.even_length_iff_even_bypass_length` : bypass length parity - `SimpleGraph.even_cycle_length_of_path` : cycle construction lemma - `SimpleGraph.bypass_eq_nil_of_closed` : closed path properties ## Proof outline 1. For bipartite graphs: use the 2-coloring to show that in a 2-coloring, a walk has even length iff its endpoints have the same color. 2. For cycles (start = end), this forces even length. 3. For the converse: if all cycles are even, construct a 2-coloring using the `two_colorable_iff_forall_loop_even` characterization. 4. Show this coloring is valid using bypass operations and path properties. ## Technical notes - Uses `SimpleGraph.Walk` for path/cycle representation - Handles both `IsPath` and `IsCycle` predicates - Uses bypass operations (`takeUntil`, `dropUntil`, `bypass`) to analyze walks - Requires `DecidableEq V` for some lemmas - Uses classical logic for case analysis ## Reviewer notes - The proof uses induction on walks and case analysis on colorings - Some lemmas (like `even_length_iff_same_color`) could be extracted to more general locations - All theorems are in the `SimpleGraph` namespace - The `bipartite_iff_all_cycles_even` theorem provides the complete characterization t-combinatorics new-contributor awaiting-author 141/5 Mathlib/Combinatorics/SimpleGraph/Bipartite.lean,Mathlib/Combinatorics/SimpleGraph/ConcreteColorings.lean 2 42 ['IvanRenison', 'NickAdfor', 'Rida-Hamadani', 'SnirBroshi', 'github-actions', 'kmill', 'mitchell-horner', 'vihdzp'] nobody
8-70778
8 days 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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR large-import 2627/30 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/Algebra/Homology/ShortComplex/ModuleCat.lean,Mathlib/Algebra/Order/Monoid/Unbundled/WithTop.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/RingTheory/CohenMacaulay/Basic.lean,Mathlib/RingTheory/CohenMacaulay/Maximal.lean,Mathlib/RingTheory/Ideal/Cotangent.lean,Mathlib/RingTheory/KrullDimension/Regular.lean,Mathlib/RingTheory/Noetherian/Basic.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 18 8 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
8-70448
8 days ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR large-import 3125/30 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/Algebra/Homology/ShortComplex/ModuleCat.lean,Mathlib/Algebra/Order/Monoid/Unbundled/WithTop.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/RingTheory/CohenMacaulay/Basic.lean,Mathlib/RingTheory/CohenMacaulay/Maximal.lean,Mathlib/RingTheory/Ideal/Cotangent.lean,Mathlib/RingTheory/KrullDimension/Regular.lean,Mathlib/RingTheory/Noetherian/Basic.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 20 8 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
8-70381
8 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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-ring-theory blocked-by-other-PR WIP 336/0 Mathlib.lean,Mathlib/RingTheory/Ideal/Cotangent.lean,Mathlib/RingTheory/RegularLocalRing/Defs.lean,Mathlib/RingTheory/RegularLocalRing/RegularRing/Basic.lean,Mathlib/RingTheory/RegularLocalRing/RegularRing/Polynomial.lean 5 4 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
8-70078
8 days ago
unknown
unknown
33032 ksenono
author:ksenono
feat(Combinatorics/SimpleGraph): Konig’s theorem on bipartite graphs --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics new-contributor blocked-by-other-PR merge-conflict 983/2 Mathlib.lean,Mathlib/Combinatorics/SimpleGraph/Basic.lean,Mathlib/Combinatorics/SimpleGraph/Bipartite.lean,Mathlib/Combinatorics/SimpleGraph/Clique.lean,Mathlib/Combinatorics/SimpleGraph/DegreeSum.lean,Mathlib/Combinatorics/SimpleGraph/Konig/Auxillary.lean,Mathlib/Combinatorics/SimpleGraph/Konig/Konig.lean,Mathlib/Combinatorics/SimpleGraph/Konig/KonigFin.lean,Mathlib/Combinatorics/SimpleGraph/Maps.lean,Mathlib/Combinatorics/SimpleGraph/Matching.lean,Mathlib/Combinatorics/SimpleGraph/Subgraph.lean,Mathlib/Combinatorics/SimpleGraph/VertexCover.lean,Mathlib/SetTheory/Cardinal/Arithmetic.lean,Mathlib/SetTheory/Cardinal/Basic.lean 14 8 ['SnirBroshi', 'github-actions', 'ksenono', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'vlad902'] nobody
8-69554
8 days ago
unknown
unknown
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` --- - [ ] depends on: #32058 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-ring-theory blocked-by-other-PR 395/0 Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Baer.lean,Mathlib/Algebra/Category/ModuleCat/Ext/DimensionShifting.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/EnoughInjectives.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/EnoughProjectives.lean,Mathlib/Algebra/Homology/ShortComplex/ModuleCat.lean,Mathlib/RingTheory/GlobalDimension.lean,Mathlib/RingTheory/Noetherian/Basic.lean 8 14 ['Thmoas-Guan', 'erdOne', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] erdOne
assignee:erdOne
8-69421
8 days ago
17-2694
17 days ago
0-341
5 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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author blocked-by-other-PR 683/0 Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Baer.lean,Mathlib/Algebra/Category/ModuleCat/Ext/DimensionShifting.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/EnoughInjectives.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/EnoughProjectives.lean,Mathlib/Algebra/Homology/ShortComplex/ModuleCat.lean,Mathlib/RingTheory/GlobalDimension.lean,Mathlib/RingTheory/LocalProperties/ProjectiveDimension.lean,Mathlib/RingTheory/Noetherian/Basic.lean 9 13 ['Thmoas-Guan', 'github-actions', 'jcommelin', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
8-69386
8 days ago
51-994
51 days ago
1-66277
1 day
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR large-import 3432/30 Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Baer.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/Algebra/Homology/ShortComplex/ModuleCat.lean,Mathlib/Algebra/Order/Monoid/Unbundled/WithTop.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/RingTheory/CohenMacaulay/Basic.lean,Mathlib/RingTheory/CohenMacaulay/Maximal.lean,Mathlib/RingTheory/GlobalDimension.lean,Mathlib/RingTheory/Ideal/Cotangent.lean,Mathlib/RingTheory/KrullDimension/Regular.lean,Mathlib/RingTheory/Noetherian/Basic.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 22 11 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
8-69321
8 days 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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR large-import 3831/30 Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Baer.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/Algebra/Homology/ShortComplex/ModuleCat.lean,Mathlib/Algebra/Order/Monoid/Unbundled/WithTop.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/RingTheory/CohenMacaulay/Basic.lean,Mathlib/RingTheory/CohenMacaulay/Maximal.lean,Mathlib/RingTheory/GlobalDimension.lean,Mathlib/RingTheory/Ideal/Cotangent.lean,Mathlib/RingTheory/KrullDimension/Regular.lean,Mathlib/RingTheory/LocalProperties/ProjectiveDimension.lean,Mathlib/RingTheory/Noetherian/Basic.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 25 12 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
8-69308
8 days 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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR large-import 2938/30 Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Baer.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/Algebra/Homology/ShortComplex/ModuleCat.lean,Mathlib/Algebra/Order/Monoid/Unbundled/WithTop.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/RingTheory/GlobalDimension.lean,Mathlib/RingTheory/Ideal/Cotangent.lean,Mathlib/RingTheory/KrullDimension/Regular.lean,Mathlib/RingTheory/Noetherian/Basic.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 20 9 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
8-69262
8 days 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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR large-import 4630/30 Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Baer.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/Algebra/Homology/ShortComplex/ModuleCat.lean,Mathlib/Algebra/Order/Monoid/Unbundled/WithTop.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/RingTheory/CohenMacaulay/Basic.lean,Mathlib/RingTheory/CohenMacaulay/Maximal.lean,Mathlib/RingTheory/GlobalDimension.lean,Mathlib/RingTheory/Ideal/Cotangent.lean,Mathlib/RingTheory/KrullDimension/Regular.lean,Mathlib/RingTheory/LocalProperties/ProjectiveDimension.lean,Mathlib/RingTheory/Noetherian/Basic.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 28 12 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
8-69231
8 days 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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR large-import WIP 4086/30 Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Baer.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/Algebra/Homology/ShortComplex/ModuleCat.lean,Mathlib/Algebra/Order/Monoid/Unbundled/WithTop.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/RingTheory/CohenMacaulay/Basic.lean,Mathlib/RingTheory/CohenMacaulay/Maximal.lean,Mathlib/RingTheory/GlobalDimension.lean,Mathlib/RingTheory/Ideal/Cotangent.lean,Mathlib/RingTheory/KrullDimension/Regular.lean,Mathlib/RingTheory/LocalProperties/ProjectiveDimension.lean,Mathlib/RingTheory/Noetherian/Basic.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 27 12 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
8-69205
8 days ago
unknown
unknown
33592 nielstron
author:nielstron
feat(Computability/ContextFreeGrammar): mapping between two types of nonterminal symbols --- This PR picks up https://github.com/leanprover-community/mathlib4/pull/15895 and resolves the failing lemma by redefining Good symbols. I checked that https://github.com/leanprover-community/mathlib4/pull/13514 builds correctly when based on this build. PR for that is #33599 This is my first contribution please let me know of any changes I should outline. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-computability new-contributor 162/0 Mathlib/Computability/ContextFreeGrammar.lean 1 1 ['github-actions', 'madvorak'] nobody
8-66767
8 days ago
9-76141
9 days ago
9-75961
9 days
32742 LTolDe
author:LTolDe
feat(MeasureTheory/Constructions/Polish/Basic): add class SuslinSpace add new class `SuslinSpace` for a topological space that is an analytic set in itself This will be useful to prove the **Effros Theorem**, see [zulip thread](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Effros.20Theorem/with/558712441). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor awaiting-zulip 4/0 Mathlib/MeasureTheory/Constructions/Polish/Basic.lean 1 9 ['ADedecker', 'LTolDe', 'dupuisf', 'github-actions', 'jcommelin'] PatrickMassot
assignee:PatrickMassot
8-65927
8 days ago
8-66080
8 days ago
11-6345
11 days
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 `#min_imports` does not give a correct set of imports. - [x] 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` blocked-by-other-PR 601/7 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
8-62947
8 days ago
unknown
unknown
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 --- - [x] depends on: #31548 - [x] depends on: #31547 - [x] depends on: #31558 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology 741/0 Mathlib.lean,Mathlib/Data/EReal/Basic.lean,Mathlib/Topology/Semicontinuity/Basic.lean,Mathlib/Topology/Sion.lean,docs/references.bib 5 8 ['AntoineChambert-Loir', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'thorimur'] dwrensha and kmill
assignee:kmill assignee:dwrensha
8-58000
8 days ago
27-34100
27 days ago
35-29821
35 days
33286 euprunin
author:euprunin
chore: golf using `grind` --- The goal of this golfing PR is to decrease the number of times lemmas are called explicitly (replacing calls to lemmas with calls to tactics). Any decrease in compilation time is a welcome side effect, although it is not a primary objective. Trace profiling results (shown if ≥10 ms before or after): * `Finset.memberSubfamily_union_nonMemberSubfamily`: 11 ms before, 116 ms after * `AkraBazziRecurrence.GrowsPolynomially.eventually_atTop_nonneg_or_nonpos`: 1181 ms before, 1194 ms after * `Equiv.Perm.support_congr`: <10 ms before, 38 ms after * `Equiv.Perm.subtypeCongr.trans`: 13 ms before, 35 ms after * `preCantorSet_antitone`: 766 ms before, 371 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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 6/28 Mathlib/Computability/AkraBazzi/GrowsPolynomially.lean,Mathlib/GroupTheory/Perm/Support.lean,Mathlib/Logic/Equiv/Basic.lean,Mathlib/Topology/Instances/CantorSet.lean 4 5 ['euprunin', 'github-actions', 'vihdzp'] thorimur
assignee:thorimur
8-52918
8 days ago
8-49482
8 days ago
20-17777
20 days
33464 Paul-Lez
author:Paul-Lez
feat(Analysis/ODE/Gronwall): Add two easy lemmas This PR adds two easy lemmas. These are the "left" version of already existing lemmas in the file. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis awaiting-author 36/0 Mathlib/Analysis/ODE/Gronwall.lean 1 2 ['github-actions', 'j-loreaux'] urkud
assignee:urkud
8-50024
8 days ago
8-50024
8 days ago
5-4419
5 days
33454 astrainfinita
author:astrainfinita
feat: lemmas about `IsometryClass` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology t-analysis awaiting-author 60/37 Mathlib/Analysis/Normed/Affine/Isometry.lean,Mathlib/Analysis/Normed/Group/Uniform.lean,Mathlib/Analysis/Normed/Operator/LinearIsometry.lean,Mathlib/Topology/MetricSpace/DilationEquiv.lean,Mathlib/Topology/MetricSpace/Isometry.lean 5 8 ['github-actions', 'j-loreaux'] urkud
assignee:urkud
8-49120
8 days ago
8-49120
8 days ago
4-41214
4 days
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) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta t-measure-probability awaiting-author 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 41 ['YaelDillies', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'thorimur', 'urkud'] RemyDegenne and thorimur
assignee:RemyDegenne assignee:thorimur
8-48412
8 days ago
unknown
unknown
32165 yuanyi-350
author:yuanyi-350
feat(Real/Trigonometric): Add `sum_cos_arith_progression` and prepare for Dirichlet kernel --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis awaiting-author merge-conflict 68/0 Mathlib.lean,Mathlib/Analysis/Fourier/DirichletKernel.lean 2 8 ['BoltonBailey', 'github-actions', 'mathlib4-merge-conflict-bot', 'urkud', 'yuanyi-350'] fpvandoorn
assignee:fpvandoorn
8-37584
8 days ago
45-24366
45 days ago
3-70866
3 days
33050 mkaratarakis
author:mkaratarakis
feat: lemmas for the analytic part of the proof of the Gelfond–Schneider theorem Lemmas missing for the formalisation of the proof of the Gelfond–Schneider theorem --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-number-theory new-contributor awaiting-author 221/0 Mathlib.lean,Mathlib/Analysis/Analytic/Basic.lean,Mathlib/Analysis/Analytic/Order.lean,Mathlib/Analysis/Complex/CauchyIntegral.lean,Mathlib/NumberTheory/Transcendental/AnalyticPart.lean 5 105 ['SnirBroshi', 'github-actions', 'j-loreaux', 'mkaratarakis', 'riccardobrasca', 'vihdzp'] riccardobrasca
assignee:riccardobrasca
8-37118
8 days ago
8-51222
8 days ago
5-6442
5 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 - [x] #31525 - [x] #31574 - [x] #31575. Claude wrote most of the text, under my prompting. 1455/1 Mathlib.lean,Mathlib/AlgebraicTopology/FundamentalGroupoid/Basic.lean,Mathlib/AlgebraicTopology/FundamentalGroupoid/SemilocallySimplyConnected.lean,Mathlib/LinearAlgebra/AffineSpace/Simplex/Centroid.lean,Mathlib/Topology/Connected/PathConnected.lean,Mathlib/Topology/Homotopy/Path.lean,Mathlib/Topology/Path.lean,Mathlib/Topology/UnitInterval.lean 8 5 ['github-actions', 'mathlib4-merge-conflict-bot'] nobody
8-33911
8 days ago
unknown
unknown
33691 kim-em
author:kim-em
feat(scripts): add find-ci-errors.sh to diagnose widespread CI failures This PR adds a script that searches through recent failed CI workflow runs to find open PRs whose current CI contains a specific error string. Useful for diagnosing widespread CI issues affecting multiple PRs (e.g., infrastructure problems, toolchain bugs). **Usage:** ```bash # Find all PRs currently failing with a specific error ./scripts/find-ci-errors.sh "Error parsing args: cannot parse arguments" # Find PRs and automatically add please-merge-master label to trigger rebuilds ./scripts/find-ci-errors.sh --please-merge-master "cannot parse arguments" ``` The `--please-merge-master` flag skips PRs with merge conflicts, and the label is automatically removed by CI once the build completes. 🤖 Prepared with Claude Code CI delegated 190/0 scripts/README.md,scripts/find-ci-errors.sh 2 4 ['bryangingechen', 'github-actions', 'mathlib-bors'] nobody
8-31616
8 days ago
8-31616
8 days ago
0-6193
1 hour
33389 khwilson
author:khwilson
feat(Mathlib/Analysis/SpecialFunctions/Log/Base): More log asymptotics A common utility in proving asymptotics is `logb b =O[⊤] log` and `(log ∘ (c * ·)) =O[atTop] log` and related lemmas `logb`. This PR fills these in for future use. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis new-contributor awaiting-author 28/2 Mathlib/Analysis/SpecialFunctions/Log/Base.lean 1 16 ['github-actions', 'j-loreaux', 'khwilson', 'vlad902'] j-loreaux
assignee:j-loreaux
8-20542
8 days ago
8-66362
8 days ago
7-54803
7 days
33368 urkud
author:urkud
feat: define `Complex.UnitDisc.shift` Also review the existing API UPD: I'm going to define a `PSL(2, Real)` action instead. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis awaiting-zulip merge-conflict 273/39 Mathlib.lean,Mathlib/Analysis/Complex/UnitDisc/Basic.lean,Mathlib/Analysis/Complex/UnitDisc/Shift.lean 3 7 ['github-actions', 'j-loreaux', 'mathlib4-merge-conflict-bot', 'sgouezel', 'urkud'] j-loreaux
assignee:j-loreaux
8-15885
8 days ago
8-62618
8 days ago
6-73017
6 days
33450 astrainfinita
author:astrainfinita
refactor: deprecate `LinearIsometryClass` --- - [ ] depends on: #33448 - [ ] depends on: #33454 This PR continues the work from #18755. Original PR: https://github.com/leanprover-community/mathlib4/pull/18755 t-algebra t-analysis blocked-by-other-PR t-topology merge-conflict
label:t-algebra$
128/125 Mathlib/Analysis/CStarAlgebra/PositiveLinearMap.lean,Mathlib/Analysis/CStarAlgebra/Spectrum.lean,Mathlib/Analysis/LocallyConvex/WeakOperatorTopology.lean,Mathlib/Analysis/Normed/Affine/Isometry.lean,Mathlib/Analysis/Normed/Algebra/Spectrum.lean,Mathlib/Analysis/Normed/Group/Uniform.lean,Mathlib/Analysis/Normed/Operator/LinearIsometry.lean,Mathlib/Topology/Algebra/Module/CharacterSpace.lean,Mathlib/Topology/Algebra/Module/Equiv.lean,Mathlib/Topology/Algebra/Module/FiniteDimension.lean,Mathlib/Topology/Algebra/Module/LinearMap.lean,Mathlib/Topology/Algebra/Module/StrongTopology.lean,Mathlib/Topology/Algebra/Module/WeakDual.lean,Mathlib/Topology/MetricSpace/DilationEquiv.lean,Mathlib/Topology/MetricSpace/Isometry.lean 15 5 ['astrainfinita', 'github-actions', 'leanprover-radar', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
8-15760
8 days ago
unknown
unknown
33295 AntoineChambert-Loir
author:AntoineChambert-Loir
feat(Algebra/Central/End): center of the group of automorphisms of a free module Let `R` be a ring and let `V` be a free `R`-module. We describe the center of the group of linear automorphisms of `V`. The group of linear automorphisms can be summoned either as `V ≃ₗ[R] V`, or as `LinearMap.GeneralLinearGroup R V`, which is a shortcut for `(V →ₗ[R] V)ˣ`. We provide both descriptions. There are three possibilities: * If `V` is trivial, then `V ≃ₗ[R] V` is trivial, and so is its center. * If `V` has rank one, then any basis with a `Unique` type of index furnishes a ring equivalence from `V →ₗ[R] V` with `Rᵐᵒᵖ`, given by right-multiplication on coordinates in the given basis. (This equivalence depends on the choice of a basis.) Then `V ≃ₗ[R] V` is mul-equivalent with `(Rᵐᵒᵖ)ˣ`, hence its center is isomorphic with `Subgroup.center (Rᵐᵒᵖ)ˣ`, or, by commutativity, with `Subgroup.center Rˣ`. * Otherwise, the center of `V ≃ₗ[R] V` consists of homotheties with central ratio, furnishing a group isomorphism from `Subgroup.center (V ≃ₗ[R] V)` with `(Subgroup.center R)ˣ`. When `R` is commutative and `V` is nontrivial, the last two cases give the same answer and the center of `V ≃ₗ[R] V` is isomorphic with `Rˣ`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra WIP
label:t-algebra$
594/0 Mathlib.lean,Mathlib/LinearAlgebra/Center.lean,Mathlib/LinearAlgebra/GeneralLinearGroup/Center.lean 3 2 ['github-actions', 'mathlib4-merge-conflict-bot'] nobody
8-3506
8 days ago
unknown
unknown
33543 JovanGerb
author:JovanGerb
feat: use `to_dual` for `HeytingAlgebra` This PR starts tagging `HeytingAlgebra` things with `to_dual`. Aligning the `Heyting` and `Coheyting` API is kind of awkward, because they are unfortunately quite different. One reason is that the arguments of `sup`/`inf` are often swapped in the dual version, which is not compatible with `to_dual`. So for now, I've done a limited amount of tagging. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 44/58 Mathlib/Combinatorics/SetFamily/Kleitman.lean,Mathlib/Order/BooleanAlgebra/Basic.lean,Mathlib/Order/Heyting/Basic.lean,Mathlib/Order/Notation.lean,Mathlib/Tactic/Translate/ToDual.lean 5 10 ['JovanGerb', 'github-actions', 'vihdzp'] nobody
7-83043
7 days ago
unknown
unknown
33702 JovanGerb
author:JovanGerb
doc(Algebra/Quotient): update `HasQuotient.Quotient` doc-string `HasQuotient.quotient'` has been deprecated (in #33037), so it should not be mentioned in the doc-string of `HasQuotent.Quotient`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra delegated
label:t-algebra$
1/6 Mathlib/Algebra/Quotient.lean 1 4 ['JovanGerb', 'github-actions', 'grunweg', 'mathlib-bors'] nobody
7-82971
7 days ago
8-4973
8 days ago
0-942
15 minutes
32583 MJ141592
author:MJ141592
refactor(SimpleGraph): change bridges not to require the edge to be present Remove the requirement for edges to exist in definition of isBridge, and then change the related lemmas to adjust for this, by renaming, fixing the statements and fixing the proofs, including in Acyclic. Closes #31690. t-combinatorics new-contributor awaiting-author 60/47 Mathlib/Combinatorics/SimpleGraph/Acyclic.lean,Mathlib/Combinatorics/SimpleGraph/Connectivity/Connected.lean 2 15 ['MJ141592', 'SnirBroshi', 'YaelDillies', 'github-actions', 'mathlib4-merge-conflict-bot'] nobody
7-73278
7 days ago
37-51741
37 days ago
0-20559
5 hours
33434 astrainfinita
author:astrainfinita
chore: redefine `Finsupp.indicator` using `Finsupp.onFinset` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data 6/17 Mathlib/Data/Finsupp/Indicator.lean 1 1 ['github-actions'] nobody
7-71250
7 days ago
10-46628
10 days ago
4-19776
4 days
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-ring-theory awaiting-author 118/0 Mathlib.lean,Mathlib/RingTheory/Ideal/Cotangent.lean,Mathlib/RingTheory/RegularLocalRing/Defs.lean 3 49 ['Thmoas-Guan', 'chrisflav', 'github-actions', 'mathlib4-merge-conflict-bot', 'mbkybky'] chrisflav
assignee:chrisflav
7-68022
7 days ago
7-73957
7 days ago
0-82130
22 hours
33192 linesthatinterlace
author:linesthatinterlace
refactor(Data/List/Induction): improve definition of `reverseRecOn` This PR improves the definition of `List.reverseRecOn`. --- This improved approach aims to give identical behavior but give a somewhat nicer proof of `List.reverseRecOn_concat`. I do not believe it is a regression in terms of performance. The approach is inspired by `biDirectionalRec`, for which I have also tweaked the definitions and proofs, albeit in a much more minor way. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data 32/27 Mathlib/Data/List/Induction.lean 1 6 ['github-actions', 'linesthatinterlace', 'vihdzp'] pechersky
assignee:pechersky
7-65445
7 days ago
7-64535
7 days ago
23-63368
23 days
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) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) delegated awaiting-CI merge-conflict 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 4 ['github-actions', 'j-loreaux', 'mathlib-bors', 'mathlib4-merge-conflict-bot'] nobody
7-60554
7 days ago
unknown
unknown
33554 themathqueen
author:themathqueen
chore(Analysis/Normed/Module/Normalize): allow for `RCLike` instead of just the reals Only the last lemma `normalize_smul` needs `ℝ`, which we rename to `normalize_real_smul`. This also makes `𝕜` explicit in half of the results. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis awaiting-author merge-conflict 67/60 Mathlib/Analysis/CStarAlgebra/Unitary/Span.lean,Mathlib/Analysis/Normed/Module/Normalize.lean,Mathlib/Geometry/Euclidean/Angle/Unoriented/Basic.lean,Mathlib/Geometry/Euclidean/Angle/Unoriented/TriangleInequality.lean,Mathlib/Geometry/Euclidean/SignedDist.lean 5 4 ['github-actions', 'j-loreaux', 'mathlib4-merge-conflict-bot', 'themathqueen'] nobody
7-59132
7 days ago
8-51881
8 days ago
1-80218
1 day
31754 dagurtomas
author:dagurtomas
feat(Topology/Category): light profinite sets are injective objects From [LeanCondensed](https://github.com/dagurtomas/LeanCondensed) --- - [ ] depends on: #32660 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology t-category-theory merge-conflict 304/0 Mathlib.lean,Mathlib/Topology/Category/LightProfinite/Injective.lean,Mathlib/Topology/Separation/Profinite.lean 3 4 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
7-48448
7 days ago
7-48449
7 days ago
1-8608
1 day
33561 kbuzzard
author:kbuzzard
chore: cont -> continuous_toFun This field is sometimes called `cont` and sometimes `continuous_toFun`. I noticed that the `continuity` tactic sometimes takes a lot longer to prove `cont` even if `continuous_toFun` is available so I thought I'd change them all to see if this speed up mathlib. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict 171/149 Mathlib/Algebra/Category/ContinuousCohomology/Basic.lean,Mathlib/Algebra/Category/ModuleCat/Topology/Homology.lean,Mathlib/Analysis/Analytic/Composition.lean,Mathlib/Analysis/Analytic/Polynomial.lean,Mathlib/Analysis/CStarAlgebra/CStarMatrix.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/NonUnital.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Unital.lean,Mathlib/Analysis/Calculus/ContDiff/FaaDiBruno.lean,Mathlib/Analysis/Calculus/FDeriv/Basic.lean,Mathlib/Analysis/Calculus/FDeriv/Extend.lean,Mathlib/Analysis/Distribution/ContDiffMapSupportedIn.lean,Mathlib/Analysis/Distribution/DerivNotation.lean,Mathlib/Analysis/Distribution/SchwartzSpace.lean,Mathlib/Analysis/Distribution/TemperedDistribution.lean,Mathlib/Analysis/Distribution/TestFunction.lean,Mathlib/Analysis/Fourier/FourierTransform.lean,Mathlib/Analysis/Fourier/LpSpace.lean,Mathlib/Analysis/InnerProductSpace/LinearPMap.lean,Mathlib/Analysis/LocallyConvex/Barrelled.lean,Mathlib/Analysis/LocallyConvex/PointwiseConvergence.lean,Mathlib/Analysis/LocallyConvex/Separation.lean,Mathlib/Analysis/LocallyConvex/WeakOperatorTopology.lean,Mathlib/Analysis/LocallyConvex/WeakSpace.lean,Mathlib/Analysis/Normed/Affine/Isometry.lean,Mathlib/Analysis/Normed/Algebra/Spectrum.lean,Mathlib/Analysis/Normed/Lp/PiLp.lean,Mathlib/Analysis/Normed/Lp/ProdLp.lean,Mathlib/Analysis/Normed/Lp/lpSpace.lean,Mathlib/Analysis/Normed/Module/Alternating/Basic.lean,Mathlib/Analysis/Normed/Module/Multilinear/Basic.lean,Mathlib/Analysis/Normed/Module/WeakDual.lean,Mathlib/Analysis/Normed/Operator/Banach.lean,Mathlib/Analysis/Normed/Operator/BoundedLinearMaps.lean,Mathlib/Analysis/Normed/Operator/Extend.lean,Mathlib/Analysis/RCLike/Extend.lean,Mathlib/Geometry/Euclidean/Incenter.lean,Mathlib/Geometry/Manifold/LocalDiffeomorph.lean,Mathlib/Geometry/Manifold/MFDeriv/Atlas.lean,Mathlib/MeasureTheory/Function/ConditionalExpectation/Basic.lean,Mathlib/MeasureTheory/Function/ConditionalExpectation/CondexpL1.lean,Mathlib/MeasureTheory/Function/SimpleFuncDenseLp.lean,Mathlib/MeasureTheory/Integral/Bochner/L1.lean,Mathlib/MeasureTheory/Measure/FiniteMeasure.lean,Mathlib/NumberTheory/ModularForms/JacobiTheta/TwoVariable.lean,Mathlib/Probability/Distributions/Fernique.lean,Mathlib/Probability/Moments/CovarianceBilinDual.lean,Mathlib/Topology/Algebra/AffineSubspace.lean,Mathlib/Topology/Algebra/Algebra.lean,Mathlib/Topology/Algebra/ContinuousAffineEquiv.lean,Mathlib/Topology/Algebra/ContinuousAffineMap.lean,Mathlib/Topology/Algebra/Module/Alternating/Basic.lean,Mathlib/Topology/Algebra/Module/Alternating/Topology.lean,Mathlib/Topology/Algebra/Module/CharacterSpace.lean,Mathlib/Topology/Algebra/Module/Equiv.lean,Mathlib/Topology/Algebra/Module/LinearMap.lean,Mathlib/Topology/Algebra/Module/LinearMapPiProd.lean,Mathlib/Topology/Algebra/Module/Multilinear/Basic.lean,Mathlib/Topology/Algebra/Module/Multilinear/Topology.lean,Mathlib/Topology/Algebra/Module/PointwiseConvergence.lean,Mathlib/Topology/Algebra/Module/Star.lean,Mathlib/Topology/Algebra/Module/StrongTopology.lean,Mathlib/Topology/Algebra/Module/WeakDual.lean,Mathlib/Topology/ContinuousMap/Algebra.lean,Mathlib/Topology/ContinuousMap/Ideals.lean,Mathlib/Topology/Instances/TrivSqZeroExt.lean,Mathlib/Topology/VectorBundle/Basic.lean 66 5 ['eric-wieser', 'github-actions', 'kbuzzard', 'leanprover-radar', 'mathlib4-merge-conflict-bot'] nobody
7-40386
7 days ago
7-40387
7 days ago
2-79879
2 days
26299 adomani
author:adomani
perf: the `commandStart` linter only acts on modified files Introduces an `IO.Ref` to allow the `commandStart` linter to only run on files that git considers modified with respect to `master`. The linter is also active on files that have had some error, as these are likely being modified! The PR should also mitigate the speed-up that the linter introduced: [#mathlib4 > A whitespace linter @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/A.20whitespace.20linter/near/525091877) Assuming that this goes well, a similar mechanism could be applied to several linters that do not need to run on all code, just on the modified code. Implementation detail: the linter is currently either on or off in "whole" files. It may be also a future development to make this more granular and only run the linter on "modifed commands in modified files", but this is not currently the plan for this modification! --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-linter awaiting-author merge-conflict 48/0 Mathlib/Tactic/Linter/CommandStart.lean 1 8 ['adomani', 'github-actions', 'grunweg', 'leanprover-bot', 'mathlib4-merge-conflict-bot'] joneugster
assignee:joneugster
7-38612
7 days ago
139-2640
139 days ago
66-67660
66 days
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) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-linter merge-conflict 84/1 Mathlib/Tactic/Linter/CommandStart.lean,MathlibTest/CommandStart.lean 2 3 ['github-actions', 'grunweg', 'mathlib4-merge-conflict-bot'] nobody
7-38069
7 days ago
unknown
unknown
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 please-adopt t-linter merge-conflict 387/19 Mathlib/Tactic/Linter/DirectoryDependency.lean,scripts/README.md,scripts/forbiddenDirs.json 3 5 ['Vierkantor', 'github-actions', 'grunweg', 'mathlib4-merge-conflict-bot'] nobody
7-35066
7 days ago
unknown
unknown
28708 sjh227
author:sjh227
feat(LinearAlgebra): define row- and column-stochastic matrices This PR defines row- and column-stochastic matrices, and relates them to doubly stochastic matrices (which are already in mathlib). --- t-data new-contributor 255/6 Mathlib.lean,Mathlib/Algebra/Group/Submonoid/Defs.lean,Mathlib/Analysis/Convex/DoublyStochasticMatrix.lean,Mathlib/LinearAlgebra/Matrix/Stochastic.lean 4 29 ['dupuisf', 'github-actions', 'j-loreaux', 'mathlib4-merge-conflict-bot', 'sjh227'] pechersky
assignee:pechersky
7-31265
7 days ago
10-43516
10 days ago
10-54841
10 days
31854 erdOne
author:erdOne
chore(AlgebraicGeometry): API for `𝒪ₓ`-modules --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebraic-geometry 430/18 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 4 ['erdOne', 'github-actions', 'joelriou', 'mathlib4-merge-conflict-bot'] dagurtomas
assignee:dagurtomas
7-31263
7 days ago
11-17975
11 days ago
11-75551
11 days
33372 kex-y
author:kex-y
feat(Probability): Countable infimum of stopping times is a stopping time --- - [x] depends on: #33371 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-measure-probability brownian 83/0 Mathlib/Probability/Process/Stopping.lean 1 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] RemyDegenne
assignee:RemyDegenne
7-31259
7 days ago
10-69420
10 days ago
10-74770
10 days
33436 astrainfinita
author:astrainfinita
feat: lemmas about `(Add)MonoidAlgebra.mapRangeRingHom` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
21/0 Mathlib/Algebra/MonoidAlgebra/Basic.lean,Mathlib/Algebra/MonoidAlgebra/MapDomain.lean 2 2 ['github-actions', 'mathlib4-merge-conflict-bot'] chrisflav
assignee:chrisflav
7-31258
7 days ago
10-44403
10 days ago
13-32694
13 days
33330 michael-novak-math
author:michael-novak-math
feat: add arc-length reparametrization of parametrized curves add new definitions of arc-length reparametrization and its corresponding parameter transformation and a theorem establishing the desired properties. t-analysis new-contributor merge-conflict 311/0 Mathlib.lean,Mathlib/Analysis/Calculus/ArcLengthReparametrization.lean,Mathlib/MeasureTheory/Integral/IntervalIntegral/FundThmCalculus.lean,docs/references.bib,lake-manifest.json 5 53 ['SnirBroshi', 'github-actions', 'grunweg', 'j-loreaux', 'mathlib4-merge-conflict-bot', 'michael-novak-math'] j-loreaux
assignee:j-loreaux
7-30246
7 days ago
7-30247
7 days ago
6-57754
6 days
33707 jcommelin
author:jcommelin
ci: add commit verification for transient and automated commits This PR adds a CI workflow that verifies PRs correctly use transient and automated commits, and provides reviewers with a clear summary of which commits need human review. Commit types: - **Substantive commits**: Regular commits requiring human review - **Automated commits** (`x: `): CI verifies the commit is the exact result of running the command on the parent - **Transient commits** (`transient: ...`): CI verifies these have zero net effect on the final tree What this PR adds: - `scripts/verify_commits.sh` - Main verification script - `scripts/verify_commits_summary.sh` - Generates PR comment from JSON output - `.github/workflows/commit_verification.yml` - GitHub Actions workflow --- ### Testing locally The commit at `HEAD^` contains test branch creation scripts. These can be used for testing the functionality of the two shell scripts. To test: ```bash # Checkout the commit with test scripts git checkout HEAD^ # Create a test branch based on your current branch (before checkout) # Save your branch name first: BASE_BRANCH=$(git rev-parse --abbrev-ref HEAD) git checkout HEAD^ ./scripts/create_test_branch.sh $BASE_BRANCH # Run verification (should pass) ./scripts/verify_commits.sh $BASE_BRANCH ./scripts/verify_commits.sh $BASE_BRANCH --json | ./scripts/verify_commits_summary.sh repo_foo 12345 # Clean up and return git checkout $BASE_BRANCH && git branch -D ci-x-test-* ``` Available test scripts: - `create_test_branch.sh` - Creates a branch with valid transient + auto commits (should pass) - `create_test_branch_fail_conflict.sh` - Transient commits cause cherry-pick conflicts (should fail) - `create_test_branch_fail_transient.sh` - Transient commits have net effect (should fail) - `create_test_branch_fail_auto.sh` - Auto commit doesn't match command output (should fail) 🤖 Generated with [Claude Code](https://claude.com/claude-code) CI merge-conflict 685/0 .github/workflows/commit_verification.yml,scripts/verify_commits.sh,scripts/verify_commits_summary.sh 3 2 ['github-actions', 'mathlib4-merge-conflict-bot'] nobody
7-27849
7 days ago
7-27850
7 days ago
0-55642
15 hours
32617 erdOne
author:erdOne
feat(RingTheory): field extension over perfect fields are smooth --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-ring-theory 150/18 Mathlib.lean,Mathlib/FieldTheory/IntermediateField/Adjoin/Algebra.lean,Mathlib/FieldTheory/IntermediateField/Adjoin/Defs.lean,Mathlib/FieldTheory/SeparableClosure.lean,Mathlib/FieldTheory/SeparablyGenerated.lean,Mathlib/RingTheory/EssentialFiniteness.lean,Mathlib/RingTheory/Smooth/Field.lean 7 6 ['chrisflav', 'erdOne', 'github-actions', 'robin-carlier'] chrisflav
assignee:chrisflav
7-25401
7 days ago
7-23881
7 days ago
17-57180
17 days
33033 kim-em
author:kim-em
feat(Tactic/Choose): add type annotation support This PR adds support for type annotations in the `choose` tactic, similar to how `intro` supports them. This allows writing: ```lean choose (n : ℕ) (hn : n > 0) using h ``` instead of just `choose n hn using h`. The type annotation is checked against the actual type from the existential, and an error is raised if they don't match. This is useful for pedagogical purposes and for catching mistakes early. Requested on Zulip: https://leanprover.zulipchat.com/#narrow/channel/187764-Lean-for-teaching/topic/adding.20type.20annotation.20to.20.60choose.60/near/564323626 🤖 Prepared with Claude Code t-meta 170/22 Mathlib/Tactic/Choose.lean,MathlibTest/choose.lean 2 20 ['AlexKontorovich', 'eric-wieser', 'fpvandoorn', 'github-actions', 'kim-em'] joneugster
assignee:joneugster
7-15073
7 days ago
7-14215
7 days ago
26-38966
26 days
33314 YuvalFilmus
author:YuvalFilmus
feat(Trigonometric/Chebyshev/Basic): calculate iterated derivatives of T and U at 1 Added theorems for the iterated derivatives of T and U at 1. These formulas are fractions, and so I also added theorems stating that the denominator divides the numerator. --- - [ ] depends on: #33312 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR 148/0 Mathlib/Analysis/SpecialFunctions/Trigonometric/Chebyshev/Basic.lean,Mathlib/RingTheory/Polynomial/Chebyshev.lean 2 4 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
6-84264
6 days ago
19-60764
19 days ago
0-882
14 minutes
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics 173/7 Mathlib/Combinatorics/SimpleGraph/CompleteMultipartite.lean 1 34 ['YaelDillies', 'b-mehta', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'mitchell-horner'] YaelDillies
assignee:YaelDillies
6-82230
6 days ago
6-81357
6 days ago
78-49490
78 days
33449 yuanyi-350
author:yuanyi-350
feat(ProbabilityTheory): Add Poisson limit theorem --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-measure-probability 145/2 Mathlib.lean,Mathlib/Probability/Distributions/Poisson.lean,Mathlib/Probability/Distributions/PoissonLimitThm.lean,docs/1000.yaml 4 4 ['github-actions', 'vihdzp'] EtienneC30
assignee:EtienneC30
6-74234
6 days ago
6-73140
6 days ago
14-3629
14 days
24010 grunweg
author:grunweg
feat(Counterexamples): a non-negative function, not a.e. zero, with vanishing lowe… …r Lebesgue integral. Came up in #23707, let's document this while we're at it. --- - [ ] depends on: #20722 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict please-adopt WIP blocked-by-other-PR t-measure-probability 110/0 Counterexamples.lean,Counterexamples/LIntegralZero.lean 2 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
6-73921
6 days ago
unknown
unknown
30855 Ruben-VandeVelde
author:Ruben-VandeVelde
fix: deprecate IsTotal in favour of Std.Total --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order merge-conflict RFC 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'] nobody
6-69843
6 days ago
57-76165
57 days ago
24-78190
24 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 6 ['SnirBroshi', 'github-actions', 'jcommelin', 'kim-em'] jcommelin
assignee:jcommelin
6-67878
6 days ago
unknown
unknown
33756 dleijnse
author:dleijnse
feat(FieldTheory): root of polynomial with p power coefficients This PR proves the results in https://stacks.math.columbia.edu/tag/031V, which gives a criterion for a root of a polynomial over a field `k` of characteristic `p` to be a `p`-th power. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra new-contributor
label:t-algebra$
88/0 Mathlib.lean,Mathlib/FieldTheory/PthPowerCoeffPoly.lean 2 1 ['github-actions'] nobody
6-67791
6 days ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict large-import t-logic 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
6-67632
6 days ago
144-45585
144 days ago
3-938
3 days
33384 sgouezel
author:sgouezel
Sg param i --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 479/12 Mathlib/Analysis/Calculus/ParametricIntegral.lean,Mathlib/Analysis/Calculus/ParametricIntervalIntegral.lean,Mathlib/MeasureTheory/Integral/DominatedConvergence.lean,Mathlib/Topology/NhdsWithin.lean,Mathlib/Topology/Separation/Regular.lean 5 3 ['github-actions', 'mathlib4-merge-conflict-bot'] nobody
6-66426
6 days ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-analysis 125/0 Mathlib/Analysis/Calculus/ParametricIntegral.lean 1 8 ['Ruben-VandeVelde', 'github-actions', 'j-loreaux', 'mathlib4-merge-conflict-bot'] j-loreaux
assignee:j-loreaux
6-62631
6 days ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR t-analysis 193/0 Mathlib/Analysis/Calculus/ParametricIntegral.lean 1 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
6-62630
6 days ago
unknown
unknown
33275 YuvalFilmus
author:YuvalFilmus
feat(Trigonometric/Chebyshev/Extremal): Chebyshev polynomials maximize iterated derivatives We prove that Chebyshev polynomials maximized iterated derivatives at points x≥1. --- - [ ] depends on: #33259 - [ ] depends on: #33274 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR 423/22 Mathlib.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Chebyshev/Extremal.lean,Mathlib/Data/Finset/Powerset.lean,Mathlib/LinearAlgebra/Lagrange.lean 4 4 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
6-59617
6 days ago
unknown
unknown
33299 kingiler
author:kingiler
feat: Add decidable membership for Interval Implemented membership and corresponding decidable instance for `Interval`. Related [#mathlib4 > Proposal: Add decidable membership for Interval](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Proposal.3A.20Add.20decidable.20membership.20for.20Interval/with/565438009). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author new-contributor t-order 16/1 Mathlib/Order/Interval/Basic.lean 1 5 ['Vierkantor', 'eric-wieser', 'github-actions', 'kingiler'] Vierkantor
assignee:Vierkantor
6-59597
6 days ago
6-59597
6 days ago
13-43705
13 days
33359 sun123zxy
author:sun123zxy
feat(Algebra/Module/SpanRank): add comparing lemmas for span rank --- Split from PR #33247 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra new-contributor
label:t-algebra$
55/6 Mathlib/Algebra/Module/SpanRank.lean 1 9 ['erdOne', 'eric-wieser', 'github-actions', 'sun123zxy'] eric-wieser
assignee:eric-wieser
6-58524
6 days ago
6-58524
6 days ago
12-55129
12 days
33274 YuvalFilmus
author:YuvalFilmus
feat(LinearAlgebra/Lagrange): Formula for iterated derivative of a polynomial using Lagrange interpolation We give a formula for the iterated derivative of a polynomial at a point using Lagrange interpolation. This will be used to prove that Chebyshev polynomials maximize iterated derivatives at points x≥1. --- - [x] depends on: #33161 - [x] depends on: #33193 - [ ] depends on: #33194 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR 106/22 Mathlib/Data/Finset/Powerset.lean,Mathlib/LinearAlgebra/Lagrange.lean 2 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
6-57542
6 days ago
unknown
unknown
32190 vihdzp
author:vihdzp
chore(Algebra/Order/Ring/Archimedean): generalize theorems to `OrderHomClass` + `RingHomClass` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
15/12 Mathlib/Algebra/Order/Hom/Ring.lean,Mathlib/Algebra/Order/Ring/Archimedean.lean 2 3 ['github-actions', 'mathlib4-merge-conflict-bot'] alreadydone
assignee:alreadydone
6-52088
6 days ago
33-45072
33 days ago
14-84289
14 days
32672 tb65536
author:tb65536
feat: haar measures on short exact sequences This PR defines the notion of a short exact sequence of topological groups, and proves that if `1 → A → B → C → 1` is a short exact sequence of topological groups, then Haar measures on `A` and `C` induce a Haar measure on `B`. The final result of the file is a consequence needed for FLT: If `B → C` is injective on an open set `U`, then `U` has bounded measure. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-measure-probability t-topology FLT 374/0 Mathlib.lean,Mathlib/MeasureTheory/Measure/Haar/Extension.lean,Mathlib/Topology/Algebra/Group/Extension.lean 3 6 ['RemyDegenne', 'github-actions', 'kbuzzard', 'tb65536'] urkud
assignee:urkud
6-46494
6 days ago
6-45533
6 days ago
35-2944
35 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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis awaiting-author merge-conflict 297/7 Mathlib/Analysis/Calculus/ParametricIntegral.lean,Mathlib/Analysis/Calculus/ParametricIntervalIntegral.lean,Mathlib/MeasureTheory/Integral/DominatedConvergence.lean,Mathlib/MeasureTheory/Integral/IntegrableOn.lean,Mathlib/Topology/NhdsWithin.lean,Mathlib/Topology/Separation/Regular.lean 6 24 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'peabrainiac', 'sgouezel'] sgouezel
assignee:sgouezel
6-45801
6 days ago
18-84662
18 days ago
11-45191
11 days
33749 plp127
author:plp127
feat: `NNRat` is countable We provide an `Encodable NNRat` instance. As a consequence we also get the instance `Countable NNRat`. See also [Zulip](https://leanprover.zulipchat.com/#narrow/channel/113489-new-members/topic/NNRat.20not.20countable.3F/near/566916284) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data large-import 13/0 Mathlib/Data/Rat/Encodable.lean 1 4 ['eric-wieser', 'github-actions', 'grunweg', 'leanprover-radar'] nobody
6-42531
6 days ago
6-39719
6 days ago
6-75554
6 days
25841 mitchell-horner
author:mitchell-horner
feat(Combinatorics/SimpleGraph): prove the Kővári–Sós–Turán theorem Prove the Kővári–Sós–Turán theorem (an upper bound on the Zarankiewicz function) --- - [x] depends on: #19865 - [x] depends on: #20738 - [x] depends on: #27602 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) --- *This PR continues the work from #20240.* *Original PR: https://github.com/leanprover-community/mathlib4/pull/20240* t-combinatorics 484/0 Mathlib.lean,Mathlib/Combinatorics/SimpleGraph/Bipartite.lean,Mathlib/Combinatorics/SimpleGraph/Extremal/KovariSosTuran.lean,Mathlib/Combinatorics/SimpleGraph/Extremal/Zarankiewicz.lean,Mathlib/Combinatorics/SimpleGraph/Maps.lean,docs/1000.yaml 6 11 ['SnirBroshi', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'mitchell-horner'] kmill
assignee:kmill
6-31259
6 days ago
10-10168
10 days ago
22-8352
22 days
33214 JJYYY-JJY
author:JJYYY-JJY
chore(Data/List/Rotate): add simp attributes * Refs #7987 (SC: Data/List/Rotate) * Add `@[simp]` to: `rotate_mod`, `rotate'_nil`, `rotate'_rotate'`, `rotate'_mod`, `rotate_rotate`, `getElem?_rotate`, `getElem_rotate`, `head?_rotate`, `map_rotate`. * Verification: `lake build Mathlib.Data.List.Rotate`. t-data new-contributor 7/0 Mathlib/Data/List/Rotate.lean 1 1 ['github-actions'] TwoFX
assignee:TwoFX
6-31255
6 days ago
23-9945
23 days ago
23-9765
23 days
33635 plp127
author:plp127
feat(Tactic/Set): use `binderIdent` instead of `ident` This let both `a` and `h` be replaced with `_` in the syntax `set a := val with ← h` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta 16/2 Mathlib/Tactic/Set.lean,MathlibTest/Set.lean 2 3 ['JovanGerb', 'github-actions', 'plp127'] kim-em
assignee:kim-em
6-31242
6 days ago
9-35211
9 days ago
9-35031
9 days
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 408/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
6-30318
6 days ago
unknown
unknown
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). t-dynamics new-contributor 757/0 Mathlib.lean,Mathlib/Dynamics/SymbolicDynamics/Basic.lean,Mathlib/Tactic/Translate/ToAdditive.lean 3 157 ['Sfgangloff', 'eric-wieser', 'github-actions', 'kckennylau', 'mathlib4-merge-conflict-bot', 'sgouezel'] sgouezel
assignee:sgouezel
6-24818
6 days ago
6-21320
6 days ago
81-45208
81 days
29203 Hagb
author:Hagb
feat(RingTheory/MvPolynomial/Groebner): add Gröbner basis This PR adds some definitions and theorems of Gröbner basis theory. 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. The previous `Mathlib/RingTheory/MvPolynomial/Groebner.lean` is moved to `Mathlib/RingTheory/MvPolynomial/Groebner/Division.lean`, and used by `Mathlib/RingTheory/MvPolynomial/Groebner/Remainder.lean` for the proof of remainder's existence. The PR is upstreamized from https://github.com/WuProver/groebner_proj. Co-authored-by: Hao Shen [3118181069@qq.com](mailto:3118181069@qq.com) --- CC @tsuki8 TODO / WIP: - [x] clean up some proofs - [x] split the file - [x] squeeze Non-terminal `simp`s - [x] add comments to explain the proof of Buchberger Criterion. - [ ] refactor something with `WithBot (σ →₀ ℕ)` variant of `MonomialOrder.degree` - [ ] refactor to use namespaces `MonomialOrder.{IsGroebnerBasis,IsRemainder}` instead of `*_of_{isGroebnerBasis,isRemainder}` in theorem names. - [ ] reduced Groebner Basis (WIP) Dependencies: - [x] depends on: #26039 S-polynomial and other lemmas in other files are split from this PR, leaving only changes of `Mathlib/RingTheory/MvPolynomial/Groebner{.lean,/*.lean}` in this PR. The following are PRs split from this PR. - [x] depends on: #32336 - [x] depends on: #32344 - [x] depends on: #32780 - [x] depends on: #32787 - [x] depends on: #32788 - [x] depends on: #32801 - [x] depends on: #32876 - [x] depends on: #32877 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-ring-theory large-import awaiting-author WIP 1649/220 Mathlib.lean,Mathlib/RingTheory/MvPolynomial/Groebner.lean,Mathlib/RingTheory/MvPolynomial/Groebner/Division.lean,Mathlib/RingTheory/MvPolynomial/Groebner/Remainder.lean,docs/references.bib 5 19 ['Hagb', 'SnirBroshi', 'erdOne', 'github-actions', 'jcommelin', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] alreadydone and erdOne
assignee:alreadydone assignee:erdOne
6-22189
6 days ago
26-27457
26 days ago
3-66580
3 days
32744 NoneMore
author:NoneMore
feat(ModelTheory/Definablity): add `DefinableFun` definition and lemmas This PR adds two basic shapes of definable sets and `DefinableFun` definition with relevant lemmas. The main result is `Set.Definable.preimage_of_map` asserting that the preimage of a definable set under a definable map is definable. There are also some tool lemmas derived by the preimage lemma. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-logic 147/0 Mathlib/ModelTheory/Definability.lean 1 59 ['NoneMore', 'github-actions', 'mathlib4-merge-conflict-bot', 'staroperator'] fpvandoorn
assignee:fpvandoorn
6-10500
6 days ago
6-8979
6 days ago
33-37831
33 days
33555 erdOne
author:erdOne
feat(RingTheory): standard smooth = etale over mvpolynomial --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import 79/2 Mathlib/Algebra/MvPolynomial/Equiv.lean,Mathlib/Algebra/MvPolynomial/PDeriv.lean,Mathlib/RingTheory/RingHom/StandardSmooth.lean 3 3 ['erdOne', 'github-actions', 'robin-carlier'] robin-carlier
assignee:robin-carlier
5-81803
5 days ago
10-50529
10 days ago
10-50349
10 days
32215 jonasvanderschaaf
author:jonasvanderschaaf
feat(ModelTheory/Types): Construct a topology on CompleteType and prove the space is TotallySeparated --- - [x] depends on: #32213 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-topology t-logic 102/0 Mathlib.lean,Mathlib/ModelTheory/Topology/Types.lean,Mathlib/ModelTheory/Types.lean,Mathlib/Tactic/Linter/DirectoryDependency.lean 4 27 ['Ruben-VandeVelde', 'Vierkantor', 'anishrajeev', 'dagurtomas', 'github-actions', 'jonasvanderschaaf', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'plp127'] dagurtomas
assignee:dagurtomas
5-73808
5 days ago
13-42587
13 days ago
15-40057
15 days
33403 xroblot
author:xroblot
feat(GroupTheory/FiniteAbelian): prove that the restriction map is surjective Let `G` be a finite commutative group and let `H` be a subgroup. If `M` is a commutative monoid such that `G →* Mˣ` and `H →* Mˣ` are both finite (this is the case for example if `M` is a commutative domain), then any homomorphism `H →* Mˣ` can be extended to an homomorphism `G →* Mˣ`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-group-theory 90/13 Mathlib/Algebra/Group/Submonoid/Operations.lean,Mathlib/GroupTheory/Exponent.lean,Mathlib/GroupTheory/FiniteAbelian/Duality.lean,Mathlib/GroupTheory/QuotientGroup/Basic.lean,Mathlib/NumberTheory/MulChar/Duality.lean,Mathlib/RingTheory/RootsOfUnity/Basic.lean 6 7 ['Ruben-VandeVelde', 'github-actions', 'xroblot'] urkud
assignee:urkud
5-69500
5 days ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology new-contributor merge-conflict 83/1 Mathlib/Topology/Baire/NonMeagre.lean,Mathlib/Topology/GDelta/Basic.lean 2 2 ['github-actions', 'mathlib4-merge-conflict-bot'] nobody
5-69281
5 days ago
104-41724
104 days ago
0-4
4 seconds
33792 xroblot
author:xroblot
feat(GroupTheory/FiniteAbelian): construct bijection between subgroups and subgroups of the dual --- - [ ] depends on: #33403 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-group-theory blocked-by-other-PR 189/16 Mathlib/Algebra/Group/Submonoid/Operations.lean,Mathlib/GroupTheory/Exponent.lean,Mathlib/GroupTheory/FiniteAbelian/Duality.lean,Mathlib/GroupTheory/QuotientGroup/Basic.lean,Mathlib/NumberTheory/MulChar/Duality.lean,Mathlib/RingTheory/RootsOfUnity/Basic.lean 6 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
5-64398
5 days ago
unknown
unknown
31925 alreadydone
author:alreadydone
feat(Topology): étalé space associated to a predicate on sections --- - [ ] depends on: #33795 migrated from #22782 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology blocked-by-other-PR 900/165 Mathlib.lean,Mathlib/AlgebraicGeometry/Modules/Tilde.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 11 15 ['adamtopaz', 'alreadydone', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] adamtopaz
assignee:adamtopaz
5-62252
5 days ago
5-62253
5 days ago
26-43791
26 days
33656 metakunt
author:metakunt
feat(Data/Nat/Choose): Add sum_range_multichoose t-data 11/0 Mathlib/Data/Nat/Choose/Sum.lean 1 6 ['eric-wieser', 'github-actions', 'metakunt'] nobody
5-62100
5 days ago
9-7156
9 days ago
9-6976
9 days
33551 metakunt
author:metakunt
feat(Data/Nat/Factorization/PrimePow): Add Nat.nontrivial_primeFactors_of_two_le_of_not_isPrimePow t-data 6/0 Mathlib/Data/Nat/Factorization/PrimePow.lean 1 4 ['Ruben-VandeVelde', 'github-actions', 'metakunt'] nobody
5-61621
5 days ago
5-61453
5 days ago
9-78323
9 days
33731 nielsvoss
author:nielsvoss
feat(Analysis/InnerProductSpace): definition of singular values for finite-dimensional inner product spaces This PR defines the singular values for linear maps between finite-dimensional inner product spaces. The API is designed in a way that allows it to be generalized to the approximation numbers, as defined in #32126. See the discussion on Zulip: https://leanprover.zulipchat.com/#narrow/channel/217875-Is-there-code-for-X.3F/topic/Singular.20Value.20Decomposition/with/558914024 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis new-contributor WIP 176/0 Mathlib/Analysis/InnerProductSpace/SingularValues.lean,docs/references.bib 2 17 ['b-mehta', 'dupuisf', 'github-actions', 'j-loreaux', 'nielsvoss', 'themathqueen'] nobody
5-57882
5 days ago
unknown
unknown
33535 erdOne
author:erdOne
feat(Algebra/Category): `Under.pushout` preserves finite limits for flat homomorphisms --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
157/5 Mathlib.lean,Mathlib/Algebra/Category/AlgCat/Basic.lean,Mathlib/Algebra/Category/AlgCat/Limits.lean,Mathlib/Algebra/Category/CommAlgCat/BaseChange.lean,Mathlib/Algebra/Category/CommAlgCat/Basic.lean,Mathlib/Algebra/Category/ModuleCat/ChangeOfRings.lean,Mathlib/Algebra/Category/ModuleCat/Limits.lean,Mathlib/Algebra/Category/Ring/Flat.lean 8 2 ['github-actions', 'robin-carlier'] eric-wieser
assignee:eric-wieser
5-55522
5 days ago
5-53830
5 days ago
11-9478
11 days
32881 foderm
author:foderm
feat(AlgebraicTopology/SimplicialObject): define simplicial homotopy This file defines the notion of a combinatorial simplicial homotopy between two morphisms of simplicial objects. A first step towards proving homotopy invariance of simplicial homotopy. See [Zulip](https://leanprover.zulipchat.com/#narrow/channel/335062-homology/topic/Homotopy.20invariance.20of.20singular.20homology/with/562221688). I left in most of my comments to make it easier to understand what indices I used, since I had to shift most of them by 1 to avoid proofs of neq 0 or similar things. I guess they can be removed once we know that the equations are the correct ones. Additionally I added some simp lemmas and an identity, I hope this is more or less how this is usually done. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebraic-topology awaiting-author 546/0 Mathlib.lean,Mathlib/AlgebraicTopology/SimplicialObject/ChainHomotopy.lean,Mathlib/AlgebraicTopology/SimplicialObject/SimplicialHomotopy.lean,Mathlib/AlgebraicTopology/SingularHomology/HomotopyInvariance.lean 4 16 ['github-actions', 'joelriou'] nobody
5-53059
5 days ago
31-45103
31 days ago
0-9663
2 hours
32856 stepan2698-cpu
author:stepan2698-cpu
feat: definition of an irreducible representation Define irreducible monoid representations over a field and prove that a monoid representation is irreducible iff the corresponding module over the monoid algebra is simple. t-algebra new-contributor
label:t-algebra$
129/10 Mathlib.lean,Mathlib/RepresentationTheory/Irreducible.lean,Mathlib/RepresentationTheory/Subrepresentation.lean 3 23 ['Whysoserioushah', 'erdOne', 'github-actions', 'stepan2698-cpu'] kim-em
assignee:kim-em
5-51787
5 days ago
5-50939
5 days ago
30-49101
30 days
33518 joelriou
author:joelriou
feat(CategoryTheory/Sites): fullness of `DescentData.pullFunctor` Let `F` be a prestack for a Grothendieck topology `J`, `f : X i ⟶ S` and `f' : X' j ⟶ S` be two families of morphisms. Assume that `f'` is a covering family for `J`, then functors `F.pullFunctor .. : F.DescentData f ⥤ F.DescentData f'` are full. (They are also faithful, but this shall be done in a separate PR #33256 where we also deduce characterizations of (pre)stacks for pretopologies.) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-category-theory 269/0 Mathlib.lean,Mathlib/CategoryTheory/Sites/Descent/Precoverage.lean 2 8 ['github-actions', 'joelriou', 'robin-carlier'] jcommelin
assignee:jcommelin
5-50356
5 days ago
5-56647
5 days ago
6-29404
6 days
30640 SnirBroshi
author:SnirBroshi
feat(Combinatorics/SimpleGraph/Acyclic): acyclic and bridge theorems --- - [x] depends on: #30542 - [x] depends on: #30570 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics 76/82 Mathlib/Combinatorics/SimpleGraph/Acyclic.lean,Mathlib/Combinatorics/SimpleGraph/Connectivity/Connected.lean 2 7 ['SnirBroshi', 'b-mehta', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] b-mehta
assignee:b-mehta
5-46365
5 days ago
5-42599
5 days ago
36-13136
36 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`. delegated t-meta merge-conflict 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 19 ['adomani', 'b-mehta', 'eric-wieser', 'github-actions', 'grunweg', 'kim-em', 'mathlib-bors', 'mathlib4-merge-conflict-bot'] nobody
5-41569
5 days ago
unknown
unknown
30579 smmercuri
author:smmercuri
feat : `v.adicCompletionIntegers K` is compact when `K` is a number field --- - [x] depends on: #30576 - [x] depends on: #33484 - [ ] depends on: #33594 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP merge-conflict blocked-by-other-PR large-import 398/20 Mathlib/NumberTheory/NumberField/FinitePlaces.lean,Mathlib/RingTheory/Valuation/Extension.lean 2 4 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
5-40142
5 days ago
unknown
unknown
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 merge-conflict 63/3 Mathlib/Tactic/Common.lean,Mathlib/Tactic/Linter/DirectoryDependency.lean,MathlibTest/canonical.lean,lake-manifest.json,lakefile.lean 5 3 ['github-actions', 'mathlib4-merge-conflict-bot'] nobody
5-40141
5 days ago
unknown
unknown
32708 morrison-daniel
author:morrison-daniel
feat(LinearAlgebra/ExteriorPower): add `Basis` for `exteriorPower` WIP --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
493/1 Mathlib.lean,Mathlib/Algebra/Module/Equiv/Basic.lean,Mathlib/LinearAlgebra/ExteriorPower/Basic.lean,Mathlib/LinearAlgebra/ExteriorPower/Basis.lean,Mathlib/LinearAlgebra/ExteriorPower/Pairing.lean,Mathlib/LinearAlgebra/LinearIndependent/Lemmas.lean,Mathlib/LinearAlgebra/PiTensorProduct/Dual.lean 7 1 ['github-actions'] nobody
5-40057
5 days ago
unknown
unknown
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 t-combinatorics new-contributor WIP merge-conflict 7725/0 Mathlib.lean,Mathlib/Analysis/Convex/SimplicialComplex/Boundary.lean,Mathlib/Combinatorics/Sperner.lean,PR_COMMENT_DRAFT.md 4 5 ['LLaurance', 'github-actions', 'mathlib4-merge-conflict-bot'] nobody
5-39785
5 days 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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR t-analysis merge-conflict 355/2 Mathlib/Analysis/Distribution/ContDiffMapSupportedIn.lean,Mathlib/Analysis/Distribution/TestFunction.lean 2 6 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
5-39783
5 days ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-analysis awaiting-author 106/2 Mathlib/Analysis/Distribution/TestFunction.lean 1 6 ['github-actions', 'j-loreaux', 'mathlib4-merge-conflict-bot'] grunweg, j-loreaux, sgouezel, urkud
assignee:urkud assignee:j-loreaux assignee:grunweg assignee:sgouezel
5-39660
5 days ago
29-46712
29 days ago
9-38808
9 days
32305 faenuccio
author:faenuccio
feat: define Sobolev Spaces Nothing to see yet. --- - [ ] depends on: #32250 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-analysis large-import blocked-by-other-PR 1812/87 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 5 ['ADedecker', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
5-39658
5 days ago
unknown
unknown
32401 ADedecker
author:ADedecker
feat: monotonicity of D^n(U) in n and in U as CLMs --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-analysis delegated 170/3 Mathlib/Analysis/Distribution/ContDiffMapSupportedIn.lean,Mathlib/Analysis/Distribution/TestFunction.lean 2 19 ['ADedecker', 'faenuccio', 'github-actions', 'j-loreaux', 'mathlib-bors', 'mathlib4-merge-conflict-bot'] nobody
5-39657
5 days ago
14-44282
14 days ago
16-51391
16 days
32410 callesonne
author:callesonne
feat(Bicategory/FunctorCategory/Pseudo): Add evaluation pseudofunctor Adding pseudofunctors `eval` and `evaluation`. WIP PR to access CI. --- - [x] depends on: #30926 - [x] depends on: #32468 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-category-theory blocked-by-other-PR 49/10 Mathlib/CategoryTheory/Bicategory/Functor/StrictlyUnitary.lean,Mathlib/CategoryTheory/Bicategory/FunctorBicategory/Pseudo.lean,Mathlib/CategoryTheory/Bicategory/Modification/Pseudo.lean,Mathlib/CategoryTheory/Bicategory/NaturalTransformation/Pseudo.lean,Mathlib/CategoryTheory/Products/Basic.lean 5 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
5-39656
5 days ago
unknown
unknown
32470 ADedecker
author:ADedecker
feat: the space of test functions is barrelled --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis merge-conflict 22/0 Mathlib/Analysis/Distribution/TestFunction.lean 1 2 ['github-actions', 'mathlib4-merge-conflict-bot'] nobody
5-39655
5 days ago
unknown
unknown
33102 adomani
author:adomani
perf: add a syntactic check for flexible linter This is very preliminary. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-linter merge-conflict 205/2 Mathlib/Tactic/Linter/FlexibleLinter.lean,MathlibTest/FlexibleLinter.lean 2 10 ['adomani', 'github-actions', 'leanprover-radar', 'mathlib4-merge-conflict-bot'] nobody
5-39529
5 days ago
unknown
unknown
33240 khwilson
author:khwilson
feat(Mathlib/Analysis/Polynomial/Norm): Introduce Polynomial.supNorm The supNorm (often called the height) of a polynomial is the max of the norm of its coefficients. Used extensively in arithmetic statistics and will support further work on counting polynomials with certain properties. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-analysis new-contributor awaiting-author 148/0 Mathlib.lean,Mathlib/Algebra/Polynomial/Coeff.lean,Mathlib/Analysis/Polynomial/MahlerMeasure.lean,Mathlib/Analysis/Polynomial/Norm.lean,Mathlib/Data/Finsupp/Basic.lean 5 48 ['MichaelStollBayreuth', 'fbarroero', 'github-actions', 'j-loreaux', 'khwilson', 'mathlib4-merge-conflict-bot', 'vihdzp'] j-loreaux
assignee:j-loreaux
5-39404
5 days ago
8-63089
8 days ago
4-76653
4 days
33645 kim-em
author:kim-em
feat(TacticAnalysis): verify grind? suggestions work This PR adds a tactic analysis linter that runs `grind?` at proof steps, captures the "Try this:" suggestions, and verifies they actually close the goal when run. Two new options: - `linter.tacticAnalysis.verifyGrind`: verify `grind?` suggestions - `linter.tacticAnalysis.verifyGrindSuggestions`: verify `grind? +suggestions` Also adds `runTacticCodeCapturingInfoTree` to capture InfoTrees during tactic execution, enabling extraction of TryThis suggestions. 🤖 Prepared with Claude Code merge-conflict t-meta 241/0 Mathlib/Lean/ContextInfo.lean,Mathlib/Tactic/TacticAnalysis.lean,Mathlib/Tactic/TacticAnalysis/Declarations.lean,MathlibTest/TacticAnalysis.lean 4 2 ['github-actions', 'mathlib4-merge-conflict-bot'] nobody
5-39272
5 days ago
unknown
unknown
33692 AntoineChambert-Loir
author:AntoineChambert-Loir
feat(LinearAlgebra/Transvection/SpecialLinearGroup): generation of the special linear group by transvections Consider transvections in the special linear group. Prove that they generate the group. Prove Dieudonné's refinement about the minimal number needed to write an element as a product of transvections. --- - [ ] depends on: #33347 - [ ] depends on: #33348 - [ ] depends on: #33387 - [ ] depends on: #33282 - [ ] depends on: #33392 - [ ] depends on: #33402 - [ ] depends on: #33485 - [ ] depends on: #32757 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra file-removed blocked-by-other-PR
label:t-algebra$
2604/222 Mathlib.lean,Mathlib/LinearAlgebra/Center.lean,Mathlib/LinearAlgebra/Determinant.lean,Mathlib/LinearAlgebra/FiniteDimensional/Lemmas.lean,Mathlib/LinearAlgebra/LinearIndependent/Lemmas.lean,Mathlib/LinearAlgebra/Transvection.lean,Mathlib/LinearAlgebra/Transvection/Basic.lean,Mathlib/LinearAlgebra/Transvection/Generation.lean,Mathlib/LinearAlgebra/Transvection/SpecialLinearGroup.lean 9 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
5-39271
5 days ago
unknown
unknown
33715 AntoineChambert-Loir
author:AntoineChambert-Loir
feat(LinearAlgebra/Projectivization/Action): prove that the action is 2-transitive and primitive Define the action of the special linear group on the projectivization. Prove that it is 2-transitive and primitive. --- - [ ] depends on: #32757 - [ ] depends on: #33387 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict file-removed blocked-by-other-PR t-algebra large-import
label:t-algebra$
1125/226 Mathlib.lean,Mathlib/LinearAlgebra/Determinant.lean,Mathlib/LinearAlgebra/FiniteDimensional/Basic.lean,Mathlib/LinearAlgebra/FiniteDimensional/Lemmas.lean,Mathlib/LinearAlgebra/Projectivization/Action.lean,Mathlib/LinearAlgebra/Projectivization/Basic.lean,Mathlib/LinearAlgebra/SpecialLinearGroup.lean,Mathlib/LinearAlgebra/Transvection.lean,Mathlib/LinearAlgebra/Transvection/Basic.lean 9 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
5-39095
5 days ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR new-contributor t-measure-probability 916/0 Mathlib.lean,Mathlib/MeasureTheory/VectorMeasure/Integral.lean,Mathlib/MeasureTheory/VectorMeasure/Variation/Defs.lean,Mathlib/MeasureTheory/VectorMeasure/Variation/Equiv.lean,Mathlib/MeasureTheory/VectorMeasure/Variation/Lemmas.lean 5 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
5-38006
5 days ago
194-1729
194 days ago
15-64852
15 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). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-data 44/10 Mathlib/Combinatorics/Derangements/Finite.lean,Mathlib/Data/Fintype/Perm.lean,Mathlib/Data/Matrix/Cartan.lean,Mathlib/LinearAlgebra/Matrix/SpecialLinearGroup.lean,MathlibTest/MatrixDetOne.lean 5 18 ['dwrensha', 'github-actions', 'leanprover-bot', 'plp127', 'robin-carlier'] robin-carlier
assignee:robin-carlier
5-36614
5 days ago
79-69999
79 days ago
12-54747
12 days
33594 smmercuri
author:smmercuri
feat: `HeightOneSpectrum.valuation` is rank one for number fields - If `K` is a number field and `v` is a height-one prime ideal then `v.valuation K` is rank one. - In general, if `v` is a rank one valuation of `K`, then its extension to the `v`-adic completion `v.Completion` is also rank one, provided in `Valuation.instRankOneCompletion` - Together these refactor and deprecate `instRankOneValuedAdicCompletion`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import 18/8 Mathlib/NumberTheory/NumberField/FinitePlaces.lean,Mathlib/RingTheory/Valuation/RankOne.lean 2 2 ['github-actions', 'smmercuri'] jcommelin
assignee:jcommelin
5-31261
5 days ago
9-73677
9 days ago
9-73497
9 days
33657 vihdzp
author:vihdzp
chore(SetTheory/Cardinal/Arithmetic): switch `lift.{max u w} x = lift.{max v w} y` to `lift.{u} x = lift.{v} y` --- Lean can't often infer the extra `w` universe otherwise. Oh, if only we had some sort of `liftEq` predicate so we didn't have to bother with `lift` at all. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-set-theory 13/13 Mathlib/SetTheory/Cardinal/Arithmetic.lean,Mathlib/SetTheory/Cardinal/Basic.lean 2 1 ['github-actions'] alreadydone
assignee:alreadydone
5-31258
5 days ago
9-6443
9 days ago
9-6263
9 days
33662 Pjotr5
author:Pjotr5
feat(Algebra/Order/BigOperators/Expect): add lemmas and strict variants ### Summary - Combine `le_expect_nonempty_of_subadditive` and `le_expect_of_subadditive` into a single lemma `le_expect_of_subadditive`. The extra assumptions `(hs : s.Nonempty)` and `(h_zero : m 0 = 0)` are unnecessary (since `m 0 = 0` follows from `h_div`). This requires a small downstream update to `Mathlib/Analysis/RCLike/Basic.lean` (`norm_expect_le`). - Add strict-inequality variants: `expect_lt_expect`, `expect_lt`, `lt_expect`. - Add existence lemmas: `exists_le_of_expect_le_expect`, `exists_le_of_le_expect`, `exists_le_of_expect_le`, and `exists_lt_of_expect_lt_expect`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor 46/16 Mathlib/Algebra/Order/BigOperators/Expect.lean,Mathlib/Analysis/RCLike/Basic.lean 2 1 ['github-actions'] dagurtomas
assignee:dagurtomas
5-31257
5 days ago
8-83692
8 days ago
8-84432
8 days
33668 Citronhat
author:Citronhat
feat(PMF): add lintegral formulas for PMF This PR introduces two lemmas describing the `lintegral` of a function with respect to the measure induced by a probability mass function: - `PMF.lintegral_eq_tsum` - `PMF.lintegral_eq_sum` These are the `ℝ≥0∞` analogues of the existing Bochner `integral` formulas `integral_eq_tsum` and `integral_eq_sum`. They could be useful for reasoning about expectations and integrability. In addition, the proof of `integral_eq_sum` is simplified by deriving it directly from `integral_eq_tsum` using `tsum_fintype`. t-measure-probability new-contributor 14/5 Mathlib/Probability/ProbabilityMassFunction/Integrals.lean 1 1 ['github-actions'] kex-y
assignee:kex-y
5-31256
5 days ago
8-35562
8 days ago
8-67060
8 days
33672 euprunin
author:euprunin
chore: golf using `grind`. add `grind` annotations. --- The goal of this golfing PR is to decrease the number of times lemmas are called explicitly (replacing calls to lemmas with calls to tactics). Any decrease in compilation time is a welcome side effect, although it is not a primary objective. Trace profiling results (shown if ≥10 ms before or after): * `Orientation.nonneg_inner_and_areaForm_eq_zero_iff_sameRay`: 287 ms before, 336 ms after * `PFunctor.liftr_iff`: 49 ms before, 93 ms after * `IsAdjoinRootMonic.coeff_root_pow`: 119 ms before, 267 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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 9/33 Mathlib/Analysis/InnerProductSpace/TwoDim.lean,Mathlib/Data/PFunctor/Univariate/Basic.lean,Mathlib/RingTheory/IsAdjoinRoot.lean 3 3 ['euprunin', 'github-actions', 'leanprover-radar'] dwrensha
assignee:dwrensha
5-31255
5 days ago
8-56754
8 days ago
8-56574
8 days
33688 Citronhat
author:Citronhat
feat(PMF): add expectation lemmas for Poisson PMF This PR adds some basic results about the Poisson distribution, its `PMF`, and its expectation. **New lemmas:** * `poissonPMF_apply` — an unfolding lemma for `poissonPMF`. * `poissonPMFReal_mul_eq_succ_mul` — the standard recursion identity for the Poisson mass function. * `poissonPMFReal_hasSum_nmul` — shows that `fun n ↦ poissonPMFReal r n * n` has sum `r`. * `poissonPMF_tsum_nmul` — the corresponding identity at the level of the `PMF`. * `poissonPMF_coe_tsum_nmul` — the same result after coercion to `ℝ`. Both `ℝ`-valued and `ℝ≥0∞`-valued formulations are included so that these results can be used conveniently in both Lebesgue and Bochner integration contexts. new-contributor t-measure-probability 21/0 Mathlib/Probability/Distributions/Poisson.lean 1 2 ['Citronhat', 'github-actions'] urkud
assignee:urkud
5-31253
5 days ago
7-41567
7 days ago
8-36876
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis new-contributor awaiting-author 70/13 Mathlib/Analysis/LocallyConvex/Separation.lean,Mathlib/Topology/Compactness/Lindelof.lean 2 43 ['ADedecker', 'CoolRmal', 'EtienneC30', 'github-actions', 'j-loreaux', 'mathlib4-merge-conflict-bot'] nobody
5-17704
5 days ago
47-73843
47 days ago
2-47050
2 days
33669 eric-wieser
author:eric-wieser
chore(Data/Nat/Digits): refactor to use List.rightpad --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import merge-conflict 32/12 Mathlib/Algebra/BigOperators/Group/List/Defs.lean,Mathlib/Algebra/Group/Basic.lean,Mathlib/Data/List/Lemmas.lean,Mathlib/Data/Nat/Digits/Defs.lean,Mathlib/Data/Nat/Digits/Lemmas.lean 5 3 ['github-actions', 'mathlib4-merge-conflict-bot', 'xroblot'] nobody
5-5246
5 days ago
unknown
unknown
32541 YaelDillies
author:YaelDillies
chore: import Tactic.Attr.Register privately This is mostly to start a discussion: Should basic tactic files like this one be re-exported by all files out of them being basic, or whether they should be explicitly imported by the few files that actually need it. Eg in #32245 Andrew and I are adding a new simp attribute, and it's a bit silly that we have to rebuild all of mathlib because that file is re-exported everywhere. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import 39/6 Mathlib/Algebra/Free.lean,Mathlib/Algebra/Group/Units/Basic.lean,Mathlib/CategoryTheory/Monoidal/Mon_.lean,Mathlib/Control/Applicative.lean,Mathlib/Control/Basic.lean,Mathlib/Control/Functor.lean,Mathlib/Control/Monad/Basic.lean,Mathlib/Control/Traversable/Basic.lean,Mathlib/Control/Traversable/Equiv.lean,Mathlib/Control/Traversable/Lemmas.lean,Mathlib/Data/Prod/Basic.lean,Mathlib/Data/Set/Operations.lean,Mathlib/Logic/Basic.lean,Mathlib/Logic/Equiv/Defs.lean,Mathlib/Logic/Function/Basic.lean,Mathlib/Logic/Function/Defs.lean,Mathlib/Logic/Nontrivial/Basic.lean,Mathlib/Tactic/Attr/Core.lean,Mathlib/Tactic/HigherOrder.lean,Mathlib/Tactic/Zify.lean 20 6 ['EtienneC30', 'YaelDillies', 'artie2000', 'github-actions', 'mathlib4-merge-conflict-bot'] kex-y
assignee:kex-y
5-785
5 days ago
38-59890
38 days ago
0-6508
1 hour
33348 AntoineChambert-Loir
author:AntoineChambert-Loir
feat(LinearAlgebra/Transvection): characterization of transvections among dilatransvections WIP. * `LinearEquiv.fixedReduce`. Pass a linear equivalence to the quotient by a fixed subspace. * Characterize transvections among dilatransvections by the fact that their reduction is the identity. --- - [ ] depends on: #33347 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra blocked-by-other-PR
label:t-algebra$
428/33 Mathlib/LinearAlgebra/Determinant.lean,Mathlib/LinearAlgebra/Transvection.lean 2 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
4-77788
4 days ago
unknown
unknown
33493 michelsol
author:michelsol
feat(RingTheory/Polynomial): An explicit formula for the Chebyshev polynomials of the first kind Adds the following explicit formula on the Chebyshev polynomial of the first kind of order n. ${ T_{n}(x)\ =\ \sum \limits _{k=0}^{\lfloor {\frac {n}{2}}\rfloor } {\binom {n}{2k}} \left(\ X^{2}-1\ \right)^{k}\ X^{n-2k}}$ This explicit formula can be found [here](https://en.wikipedia.org/wiki/Chebyshev_polynomials#Explicit_expressions). There is a proof using complex numbers but it only works if the ring R = ℂ. The proof here is by induction and works in a commutative ring R. Mathlib seems to extend the definition of Chebyshev polynomials for $n \in \mathbb{Z}$ but this would make the formula more cumbersome with `n.natAbs` in place of `n`'s, so I expressed it on `n : ℕ` directly. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-ring-theory new-contributor 51/1 Mathlib/RingTheory/Polynomial/Chebyshev.lean 1 8 ['YuvalFilmus', 'erdOne', 'github-actions', 'metakunt', 'michelsol'] erdOne
assignee:erdOne
4-67693
4 days ago
10-53211
10 days ago
11-43702
11 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.isEffective_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 awaiting-author t-ring-theory 214/1 Mathlib.lean,Mathlib/LinearAlgebra/TensorProduct/Tower.lean,Mathlib/RingTheory/TensorProduct/IncludeLeftSubRight.lean,Mathlib/RingTheory/TensorProduct/Maps.lean 4 28 ['erdOne', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'yonggyuchoimath'] PatrickMassot and erdOne
assignee:PatrickMassot assignee:erdOne
4-67319
4 days ago
4-67319
4 days ago
56-62025
56 days
33604 xgenereux
author:xgenereux
feat(ValuationSubring): eq_top_iff + qol changes Given a `A : ValuationSubring K`, this PR adds the lemma `eq_top_iff : A = ⊤ ↔ ¬ A.valuation.IsNontrivial`. I have also made some small quality of life changes: 1. Added other forms of the basic rewrite lemmas with `Valuation.IsEquiv`: - `eq_zero` - `one_le_iff_one_le` - ~~`neq_one_iff_neq_one`~~ - `one_lt_iff_one_lt` - removed : `ne_zero` 2. Reorganized section following the `IsEquiv` namespace block in Valuation.Basic 3. Added lemmas `(h : v.IsEquiv v') : v.IsNontrivial ↔ v'.IsNontrivial` - `isNontrivial_of_isEquiv` - `isNontrivial_iff_isEquiv_isNontrivial` 4. Added simp tags 5. Added simp lemmas - `isNontrivial_valuationSubring_valuation_iff` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-ring-theory 69/38 Mathlib/NumberTheory/Padics/ValuativeRel.lean,Mathlib/RingTheory/Valuation/Basic.lean,Mathlib/RingTheory/Valuation/ValuationSubring.lean,Mathlib/RingTheory/Valuation/ValuativeRel/Basic.lean,Mathlib/Topology/Algebra/Valued/WithVal.lean 5 22 ['erdOne', 'github-actions', 'mathlib4-merge-conflict-bot', 'vihdzp', 'xgenereux'] nobody
4-58196
4 days ago
4-64352
4 days ago
4-55008
4 days
33612 xgenereux
author:xgenereux
feat(ValuationSubring): fieldTop Given a field `K`, the top element of `ValuationSubring K` is `K`, so top is also a field. Note: I fear this would be a bad instance so I have marked this as an abbrev for now. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-ring-theory 4/0 Mathlib/RingTheory/Valuation/ValuationSubring.lean 1 8 ['erdOne', 'github-actions', 'vihdzp', 'xgenereux'] mattrobball
assignee:mattrobball
4-57377
4 days ago
4-56442
4 days ago
9-46555
9 days
31795 thorimur
author:thorimur
feat: turn on `unusedFintypeInType` linter This PR turns on the `unusedFintypeInType` linter introduced in #31794 by adding it to the `mathlibStandardSet` of linters in Mathlib.Init. --- - [ ] depends on: #31794 - [x] depends on: #33068 - [x] depends on: #33148 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR merge-conflict file-removed 311/46 Mathlib/Data/Fintype/EquivFin.lean,Mathlib/Data/Fintype/Quotient.lean,Mathlib/Init.lean,Mathlib/Tactic/Linter/UnusedInstancesInType.lean,MathlibTest/UnusedInstancesInType/Basic.lean,MathlibTest/UnusedInstancesInType/Decidable.lean,MathlibTest/UnusedInstancesInType/Fintype.lean,MathlibTest/UnusedInstancesInType/FintypeNeedingImport.lean,MathlibTest/UnusedInstancesInType/SetOption.lean 9 10 ['SnirBroshi', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'thorimur'] nobody
4-53876
4 days ago
unknown
unknown
33049 xgenereux
author:xgenereux
feat: Valuation.IsTrivialOn A valuation on an `A`-algebra `B` is trivial on constants if the nonzero elements of the base ring `A` are mapped to `1`. ``` variable {Γ₀ : Type*} [LinearOrderedCommGroupWithZero Γ₀] class IsTrivialOn {B : Type*} (A : Type*) [CommSemiring A] [Ring B] [Algebra A B] (v : Valuation B Γ₀) where eq_one : ∀ a : A, a ≠ 0 → v (algebraMap A B a) = 1 ``` This is true, for example, when `A` is a finite field. See `Valuation.FiniteField.instIsTrivialOn`. See discussion in PR #30505 [here](https://github.com/leanprover-community/mathlib4/pull/30505#discussion_r2482320357). Note: The property could also be named `IsTrivialOn.trivial` or `IsTrivialOn.eq_one₀` instead of `trivial`. Let me know what you prefer. Co-authored-by: María Inés de Frutos Fernández <[mariaines.dff@gmail.com](mailto:mariaines.dff@gmail.com)> --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-ring-theory 71/0 Mathlib.lean,Mathlib/GroupTheory/OrderOfElement.lean,Mathlib/RingTheory/Valuation/Basic.lean,Mathlib/RingTheory/Valuation/FiniteField.lean 4 16 ['erdOne', 'github-actions', 'xgenereux'] nobody
4-42202
4 days ago
11-46557
11 days ago
1-44483
1 day
33658 vihdzp
author:vihdzp
refactor(RingTheory/Valuation/ValuativeRel/Basic): fix theorem names for multiplication We rename `vle_mul_right` to `mul_vle_mul_left` and reorder its arguments to match `mul_le_mul_left`, and other analogous changes. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-ring-theory 63/64 Mathlib/RingTheory/Valuation/ValuativeRel/Basic.lean,Mathlib/RingTheory/Valuation/ValuativeRel/Trivial.lean 2 7 ['JovanGerb', 'erdOne', 'github-actions'] erdOne
assignee:erdOne
4-38512
4 days ago
4-36882
4 days ago
8-73320
8 days
25905 mans0954
author:mans0954
feat(RingTheory/Polynomial/SmallDegreeVieta): polynomial versions of results in Algebra.QuadraticDiscriminant This PR continues the work from #25605. Original PR: https://github.com/leanprover-community/mathlib4/pull/25605 merge-conflict t-ring-theory please-adopt 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
4-38184
4 days ago
130-66563
130 days ago
81-61193
81 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 please-adopt
label:t-algebra$
182/0 Mathlib/Algebra/CharP/Invertible.lean,Mathlib/RingTheory/RootsOfUnity/Complex.lean 2 3 ['github-actions', 'mans0954', 'urkud'] jcommelin
assignee:jcommelin
4-38167
4 days ago
56-51752
56 days ago
156-74678
156 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 merge-conflict WIP t-analysis large-import please-adopt 377/3 Mathlib/Analysis/LocallyConvex/AbsConvex.lean,Mathlib/Analysis/LocallyConvex/Polar.lean,Mathlib/Analysis/Normed/Module/WeakDual.lean,Mathlib/Topology/UniformSpace/Cauchy.lean 4 5 ['github-actions', 'mans0954', 'mathlib4-merge-conflict-bot'] nobody
4-38145
4 days ago
unknown
unknown
26340 mans0954
author:mans0954
feat(Algebra/Module/NestAlgebra): Nest algebras This PR continues the work from #18705. Original PR: https://github.com/leanprover-community/mathlib4/pull/18705 merge-conflict t-algebra please-adopt
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
4-38129
4 days ago
unknown
unknown
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 WIP t-algebra please-adopt
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 2 ['github-actions', 'mans0954'] nobody
4-38121
4 days ago
unknown
unknown
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 merge-conflict WIP t-algebra large-import please-adopt
label:t-algebra$
888/0 Mathlib.lean,Mathlib/Data/Sym/Sym2/Prod.lean,Mathlib/LinearAlgebra/QuadraticForm/Basis.lean 3 3 ['github-actions', 'mans0954', 'mathlib4-merge-conflict-bot'] nobody
4-37898
4 days ago
unknown
unknown
26343 mans0954
author:mans0954
feat(Analysis/Normed/Module/Complemented): The idempotent associated with a complemented subspace Given a complemented subspace `p` of a Banach space `E`, with complement `q`, there exists an idempotent `P` in the ring `E →L[𝕜] E` such that `P` has range `p` and kernel `q`. Similarly `1-P` has range `q` and kernel `p`. See Rudin, Functional Analysis, Theorem 5.16. --- This PR continues the work from #20330. Original PR: https://github.com/leanprover-community/mathlib4/pull/20330 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP awaiting-CI large-import merge-conflict t-analysis please-adopt 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
4-37891
4 days ago
unknown
unknown
33808 seewoo5
author:seewoo5
feat(Manifold/MFDeriv): add fun_prop to `MDifferentiable` --- Add FunProp to `MDifferentiable`. For example, the following works (when `F'` is normed `𝕜`-algebra) ```lean example (hp : MDifferentiable I 𝓘(𝕜, F') p) (hq : MDifferentiable I 𝓘(𝕜, F') q) : MDifferentiable I 𝓘(𝕜, F') ((p * q + p - q) * q * p) := by fun_prop ``` Motivated from [sphere packing project](https://github.com/thefundamentaltheor3m/Sphere-Packing-Lean). [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-differential-geometry 15/0 Mathlib/Geometry/Manifold/MFDeriv/Basic.lean,Mathlib/Geometry/Manifold/MFDeriv/Defs.lean,Mathlib/Geometry/Manifold/MFDeriv/SpecificFunctions.lean 3 8 ['github-actions', 'grunweg', 'seewoo5'] nobody
4-33493
4 days ago
5-3576
5 days ago
0-39986
11 hours
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 merge-conflict WIP t-analysis file-removed please-adopt 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
4-32694
4 days ago
unknown
unknown
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 merge-conflict awaiting-author t-analysis large-import please-adopt 322/64 Mathlib/Analysis/LocallyConvex/AbsConvex.lean,Mathlib/Analysis/LocallyConvex/Bipolar.lean,Mathlib/Analysis/LocallyConvex/Polar.lean,Mathlib/Analysis/LocallyConvex/WeakDual.lean,Mathlib/Topology/Algebra/Module/LinearSpan.lean,Mathlib/Topology/Algebra/Module/StrongTopology.lean,Mathlib/Topology/Algebra/Module/WeakBilin.lean 7 110 ['JonBannon', 'eric-wieser', 'faenuccio', 'github-actions', 'j-loreaux', 'leanprover-community-bot-assistant', 'mans0954', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'mcdoll'] faenuccio and j-loreaux
assignee:j-loreaux assignee:faenuccio
4-32689
4 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 merge-conflict WIP t-algebra please-adopt
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
4-32675
4 days ago
unknown
unknown
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 merge-conflict t-data please-adopt 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
4-32671
4 days ago
57-6769
57 days ago
142-36931
142 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 help-wanted t-analysis please-adopt 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
4-32627
4 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 merge-conflict WIP t-analysis please-adopt 125/0 Mathlib.lean,Mathlib/Analysis/LocallyConvex/Prime.lean 2 3 ['github-actions', 'mans0954', 'mathlib4-merge-conflict-bot'] nobody
4-32618
4 days ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-order please-adopt 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
4-32585
4 days ago
101-56842
101 days ago
0-19323
5 hours
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict please-adopt 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
4-32552
4 days ago
57-5506
57 days ago
41-43711
41 days
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR t-analysis please-adopt 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
4-32533
4 days ago
130-56864
130 days ago
0-5
5 seconds
30393 mans0954
author:mans0954
WIP: Bipolar theorem absconvex refactor Experiment to see what happens when #26345 and #29342 are merged. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP large-import please-adopt 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 2 ['github-actions', 'mathlib4-merge-conflict-bot'] nobody
4-32389
4 days 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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-analysis please-adopt 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
4-32373
4 days ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis please-adopt 110/11 Mathlib/Analysis/Normed/Ring/Basic.lean,MathlibTest/TCSynth.lean 2 15 ['github-actions', 'j-loreaux', 'leanprover-bot'] ADedecker
assignee:ADedecker
4-32291
4 days ago
57-41944
57 days ago
57-10323
57 days
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 merge-conflict WIP t-analysis large-import please-adopt 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 4 ['github-actions', 'mans0954', 'mathlib4-merge-conflict-bot'] nobody
4-32114
4 days ago
unknown
unknown
26614 Rida-Hamadani
author:Rida-Hamadani
feat(SimpleGraph): add more API for `take`/`drop` 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`, alongside a similar lemma for dropping vertices. --- - [x] depends on: #26655 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics 58/0 Mathlib/Combinatorics/SimpleGraph/Walks/Operations.lean,Mathlib/Combinatorics/SimpleGraph/Walks/Subwalks.lean 2 20 ['Rida-Hamadani', 'b-mehta', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] kmill
assignee:kmill
4-31244
4 days ago
23-25219
23 days ago
28-18879
28 days
33611 urkud
author:urkud
feat(ImplicitFunction): add a parametric version --- I'm not sure if the supporting linear algebra lemmas are in the form we want to see them in Mathlib. - [x] depends on: #33585 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis 191/0 Mathlib.lean,Mathlib/Analysis/Calculus/FDeriv/Prod.lean,Mathlib/Analysis/Calculus/ImplicitFunction/Parametric.lean,Mathlib/LinearAlgebra/Prod.lean 4 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] ADedecker
assignee:ADedecker
4-31239
4 days ago
8-10634
8 days ago
9-46420
9 days
33649 vihdzp
author:vihdzp
feat(Analysis/Real/Hyperreal): more lemmas on `ω` and `ε` I've moved these around a bit, so as to ensure the lemmas about each constant are next to each other. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-algebra
label:t-algebra$
116/30 Mathlib/Algebra/Order/AddGroupWithTop.lean,Mathlib/Algebra/Order/Ring/Archimedean.lean,Mathlib/Algebra/Order/Ring/StandardPart.lean,Mathlib/Analysis/Real/Hyperreal.lean 4 6 ['github-actions', 'vihdzp', 'wwylele'] kim-em
assignee:kim-em
4-31237
4 days ago
9-13883
9 days ago
9-13703
9 days
33700 vihdzp
author:vihdzp
feat: dense orders have elements lying between two finite sets Used in the CGT repo, and will be used not too long in the future to show dense orders are η₀-sets. Co-authored-by: Kenny Lau --- See [Zulip](https://leanprover.zulipchat.com/#narrow/channel/217875-Is-there-code-for-X.3F/topic/.60exists_between.60.20for.20finite.20sets/near/526965677). Is the import increase a problem? If so, would a new file for these theorems be desirable? Or where else should they go? [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order large-import 30/0 Mathlib/Data/Finset/Max.lean 1 1 ['github-actions'] Vierkantor
assignee:Vierkantor
4-31232
4 days ago
8-15413
8 days ago
8-15233
8 days
33724 alreadydone
author:alreadydone
chore(Algebra): deprecate `DistribMulAction.toAddMonoidHom` which is simply a specialized version of `DistribSMul.toAddMonoidHom`. `MulDistribMulAction.toMonoidHom` has to be kept, since there is no `MulDistribSMul` yet. also deprecate `AddMonoidHom.smulLeft` (same situation) and generalize `DistribMulAction.toLinearMap` --- - [x] depends on: #33721 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
111/99 Mathlib/Algebra/Algebra/Hom.lean,Mathlib/Algebra/Algebra/Tower.lean,Mathlib/Algebra/BigOperators/Finprod.lean,Mathlib/Algebra/Category/ModuleCat/Tannaka.lean,Mathlib/Algebra/DirectSum/Algebra.lean,Mathlib/Algebra/GroupWithZero/Action/Basic.lean,Mathlib/Algebra/GroupWithZero/Action/Defs.lean,Mathlib/Algebra/GroupWithZero/Action/End.lean,Mathlib/Algebra/Module/Basic.lean,Mathlib/Algebra/Module/Equiv/Basic.lean,Mathlib/Algebra/Module/Hom.lean,Mathlib/Algebra/Module/LinearMap/Defs.lean,Mathlib/Algebra/Module/LinearMap/End.lean,Mathlib/Algebra/Module/Rat.lean,Mathlib/Algebra/Module/Submodule/Invariant.lean,Mathlib/Algebra/Module/Submodule/Pointwise.lean,Mathlib/Algebra/Module/Torsion/Basic.lean,Mathlib/Algebra/Polynomial/HasseDeriv.lean,Mathlib/Algebra/QuadraticAlgebra/NormDeterminant.lean,Mathlib/Algebra/Ring/Action/Basic.lean,Mathlib/Analysis/SpecialFunctions/Gamma/BohrMollerup.lean,Mathlib/LinearAlgebra/AffineSpace/Pointwise.lean,Mathlib/LinearAlgebra/BilinearMap.lean,Mathlib/LinearAlgebra/Matrix/ToLin.lean,Mathlib/LinearAlgebra/TensorProduct/Basic.lean,Mathlib/LinearAlgebra/TensorProduct/Graded/External.lean,Mathlib/RingTheory/DiscreteValuationRing/TFAE.lean,Mathlib/RingTheory/FractionalIdeal/Basic.lean,Mathlib/RingTheory/IntegralClosure/Algebra/Basic.lean,Mathlib/RingTheory/Jacobson/Ideal.lean,Mathlib/RingTheory/Morita/Matrix.lean,Mathlib/RingTheory/Regular/IsSMulRegular.lean,Mathlib/Topology/Algebra/InfiniteSum/Module.lean,Mathlib/Topology/Algebra/Ring/Real.lean,Mathlib/Topology/Algebra/UniformMulAction.lean 35 2 ['github-actions', 'mathlib4-dependent-issues-bot'] jcommelin
assignee:jcommelin
4-31230
4 days ago
7-39588
7 days ago
7-39408
7 days
33501 SnirBroshi
author:SnirBroshi
feat(Combinatorics/SimpleGraph/Finite): degrees for infinite graphs - Redefine degrees using `Set.ncard` to avoid `Fintype` and enable talking about degrees in infinite graphs. - Define `ENat` versions of `degree`/`minDegree`/`maxDegree` called `edegree`/`eminDegree`/`emaxDegree` respectively. - Remove `LocallyFinite` assumption from `IsRegularOfDegree`, and change it to use `edegree = k` instead of `degree = k` to retain the meaning of the case `k = 0`. --- The `e` prefix matches the existing `edist` and `ediam`. To make reviewing easier, this PR intentionally does not: - Add theorems about the new definitions - Reorder theorems to avoid `omit`s - Move theorems to a new `Degree.lean` file This is so that the diff shows the old/new versions side-by-side, and to avoid a bigger PR. Consequently a few proofs are a bit longer, but that'll be fixed after this PR by adding API lemmas for the new definitions (e.g. `edegree ≠ ⊤ → edegree = degree`). Regarding computability: If computability of degrees is useful, we can introduce a separate `findegree` in the future (similar to `neighborSet` vs `neighborFinset`), but I think degrees are a basic graph definition that should be defined for any `SimpleGraph`. As for theorems, such a `findegree` can use a lemma `findegree = degree` to access all the degree theorems, instead of duplicating everything to both versions. This PR was motivated by wanting to talk about infinite graphs with a finite max-degree. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-combinatorics 302/243 Archive/Wiedijk100Theorems/FriendshipGraphs.lean,Archive/Wiedijk100Theorems/Konigsberg.lean,Counterexamples/HeawoodUnitDistance.lean,Mathlib/Combinatorics/SimpleGraph/Acyclic.lean,Mathlib/Combinatorics/SimpleGraph/AdjMatrix.lean,Mathlib/Combinatorics/SimpleGraph/Bipartite.lean,Mathlib/Combinatorics/SimpleGraph/Circulant.lean,Mathlib/Combinatorics/SimpleGraph/Connectivity/Connected.lean,Mathlib/Combinatorics/SimpleGraph/DegreeSum.lean,Mathlib/Combinatorics/SimpleGraph/Extremal/Turan.lean,Mathlib/Combinatorics/SimpleGraph/Finite.lean,Mathlib/Combinatorics/SimpleGraph/FiveWheelLike.lean,Mathlib/Combinatorics/SimpleGraph/LapMatrix.lean,Mathlib/Combinatorics/SimpleGraph/Maps.lean,Mathlib/Combinatorics/SimpleGraph/Prod.lean,Mathlib/Combinatorics/SimpleGraph/StronglyRegular.lean,Mathlib/Combinatorics/SimpleGraph/Subgraph.lean,Mathlib/Combinatorics/SimpleGraph/Trails.lean,Mathlib/Data/Set/Card.lean,Mathlib/Data/Set/Insert.lean,Mathlib/Order/ConditionallyCompleteLattice/Finset.lean 21 1 ['github-actions'] nobody
4-31154
4 days ago
11-62192
11 days ago
11-62012
11 days
33665 JovanGerb
author:JovanGerb
fix(addRelatedDecl): support imported theorems in module This PR lets `elementwise`, `to_fun`, etc. work on theorems that are imported (and the body of the theorem is not available). These kinds of declarations have the axiom constant info, which was not supported before. As a bonus, I've also made it support unsafe theorems. I've removed the support for the auxiliary declaration being a `def`, because this is never used, and it wasn't clear to me what the expected behaviour there is exactly (e.g. should it be `reducible`?). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta 3/18 Mathlib/CategoryTheory/ConcreteCategory/Elementwise.lean,Mathlib/CategoryTheory/Elementwise.lean,Mathlib/Util/AddRelatedDecl.lean 3 2 ['adamtopaz', 'github-actions'] adamtopaz
assignee:adamtopaz
4-30693
4 days ago
8-69011
8 days ago
8-68831
8 days
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'` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-zulip t-logic 78/72 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,Mathlib/RingTheory/Congruence/Hom.lean 8 9 ['SnirBroshi', 'github-actions', 'mathlib4-merge-conflict-bot', 'thorimur', 'vihdzp'] thorimur
assignee:thorimur
4-25106
4 days ago
84-31824
84 days ago
8-45935
8 days
33209 JovanGerb
author:JovanGerb
feat(infoview_search): move to new frontend This PR changes the UI of `#infoview_search`, so that the replacement expression is hoverable, and there is a separate insert button. I posted screenshots in [#mathlib4 > `rw??` discussion @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/.60rw.3F.3F.60.20discussion/near/565081431) --- - [ ] depends on: #33052 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import file-removed t-meta blocked-by-other-PR 191/108 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Common.lean,Mathlib/Tactic/InfoviewSearch/InteractiveUnfold.lean,Mathlib/Tactic/InfoviewSearch/LibraryRewrite.lean,Mathlib/Tactic/InfoviewSearch/Util.lean,MathlibTest/LibraryRewrite.lean 7 4 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
4-23047
4 days ago
unknown
unknown
33052 JovanGerb
author:JovanGerb
feat: replace `rw??` tactic with `#infoview_search` command This PR introduces the `#infoview_search` command. It gives an improved way of interacting with the library search from `rw??`, and hence this PR also deprecates `rw??` (`rw??` still works, but it displays a warning message suggesting to use `#infoview_search` instead). The difference is that `#infoview_search` is a command, so you type it once, and then you can use rewrite search in any tactic state in any place. This is more convenient than having to write out `rw??` every time. I have many improvements planned for `#infoview_search`, but this PR simply gives it the same capabilities that `rw??` currently has. One of those improvements is to also do `apply` search, and `apply at` search. That is why the name doesn't contain `rw` anymore. To prepare for more code developments around `#infoview_search`, I've moved the relevant files into a new folder `Mathlib.Tactic.InfoviewSearch`. Note that one annoyance with writing `#infoview_search` is that there is a linter warning. Should I remove the `#` from the command, or are we happy with this? ``` `#`-commands, such as '#infoview_search', are not allowed in 'Mathlib' Note: This linter can be disabled with `set_option linter.hashCommand false` ``` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-meta file-removed 100/59 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Common.lean,Mathlib/Tactic/InfoviewSearch/InteractiveUnfold.lean,Mathlib/Tactic/InfoviewSearch/LibraryRewrite.lean,MathlibTest/LibraryRewrite.lean 6 2 ['github-actions', 'mathlib4-merge-conflict-bot'] adamtopaz
assignee:adamtopaz
4-22367
4 days ago
5-39531
5 days ago
21-82457
21 days
33025 JovanGerb
author:JovanGerb
feat(gcongr): beef up `@[gcongr]` tag to accept `↔` & any argument order This PR modifies the `@[gcongr]` tag to accept lemmas in more forms. - Iff lemmas are now accepted, and are turned into an auxiliary lemmas that is simply one of the two implications. - Implicational gcongr lemmas now don't need to have their arguments given in the "correct" order. An auxiliary lemma is generated if necessary. The auxiliary lemma generation is done analogously to `simp` which creates little lemmas `Foo._simp_1`., I also went throught all lemmas that have `GCongr.` in the name, and removed all but one of them (the remaining one is `GCongr.mem_of_le_of_mem`) A future PR may introduce the `gcongr at` tactic, which does `gcongr` but at hypotheses. This would be using the reverse direction of the iff lemmas tagged with `gcongr`. For this reason it is preferred to tag the iff lemma if possible. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta 208/278 Mathlib/Algebra/Module/Submodule/Basic.lean,Mathlib/Algebra/Order/BigOperators/Expect.lean,Mathlib/Algebra/Order/Pi.lean,Mathlib/Algebra/Order/Ring/Cast.lean,Mathlib/Algebra/Order/Ring/Ordering/Basic.lean,Mathlib/Analysis/SpecialFunctions/Arsinh.lean,Mathlib/Data/Finset/Defs.lean,Mathlib/Data/Finset/Image.lean,Mathlib/Data/Finset/Range.lean,Mathlib/Data/Finsupp/Order.lean,Mathlib/Data/Int/Basic.lean,Mathlib/Data/NNReal/Defs.lean,Mathlib/Data/Set/Insert.lean,Mathlib/Data/SetLike/Basic.lean,Mathlib/MeasureTheory/Function/SimpleFunc.lean,Mathlib/NumberTheory/LucasLehmer.lean,Mathlib/Order/Basic.lean,Mathlib/Order/Filter/Basic.lean,Mathlib/Order/Fin/Basic.lean,Mathlib/Order/Hom/Basic.lean,Mathlib/Order/Hom/Lattice.lean,Mathlib/Order/Interval/Finset/Basic.lean,Mathlib/Order/Interval/Set/Basic.lean,Mathlib/Order/Nucleus.lean,Mathlib/Order/Sublocale.lean,Mathlib/RingTheory/FractionalIdeal/Basic.lean,Mathlib/SetTheory/ZFC/VonNeumann.lean,Mathlib/Tactic/GCongr/Core.lean,Mathlib/Tactic/Translate/Core.lean,MathlibTest/GCongr/GCongr.lean 30 3 ['github-actions', 'mathlib4-merge-conflict-bot'] dwrensha
assignee:dwrensha
4-22195
4 days ago
4-17201
4 days ago
27-16902
27 days
33507 khwilson
author:khwilson
feat(Mathlib/Analysis/Polynomial/Fourier): Add Parseval's Identity specialized to Polynomials Parseval's identity specialized to polynomials states that the sum of the norm squared coefficients is equal to the average of the norm of the polynomial squared on the circle. We prove this fact. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis new-contributor awaiting-author 181/0 Mathlib.lean,Mathlib/Analysis/Complex/Circle.lean,Mathlib/Analysis/Fourier/AddCircle.lean,Mathlib/Analysis/Polynomial/Fourier.lean,Mathlib/Analysis/SpecialFunctions/Complex/Circle.lean 5 16 ['adomani', 'eric-wieser', 'github-actions', 'j-loreaux', 'khwilson'] nobody
4-19464
4 days ago
8-46036
8 days ago
3-17908
3 days
33815 grunweg
author:grunweg
style: fix whitespace around conditional variance The majority of cases in mathlib uses no space around the pipes, so do the same here. This matches how the notation pretty-prints. Found by extending the whitespace linter to proof bodies in #30658. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-measure-probability awaiting-author 39/39 Mathlib/Probability/CondVar.lean,Mathlib/Probability/Independence/Conditional.lean 2 4 ['Komyyy', 'RemyDegenne', 'github-actions', 'grunweg'] nobody
4-3567
4 days ago
4-3567
4 days ago
0-82782
22 hours
33417 themathqueen
author:themathqueen
feat: `{Continuous}Linear{Isometry}Equiv.conj{Continuous, Star}AlgEquiv` are "almost" injective ... "almost" meaning that they are colinear. I.e., `f.conj{Continuous, Star}AlgEquiv S = g.conj{Continuous, Star}AlgEquiv S` iff `f = α • g` for some (unitary) `α`. Also, the same for `Unitary.conjStarAlgAut`. All in one PR since they all have analogous proofs. --- - [x] depends on: #33301 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis t-algebra
label:t-algebra$
243/4 Mathlib/Algebra/Central/End.lean,Mathlib/Algebra/Module/Equiv/Defs.lean,Mathlib/Algebra/Star/UnitaryStarAlgAut.lean,Mathlib/Analysis/InnerProductSpace/Adjoint.lean,Mathlib/Analysis/Normed/Operator/ContinuousAlgEquiv.lean,Mathlib/Topology/Algebra/Module/Equiv.lean 6 6 ['github-actions', 'mathlib4-dependent-issues-bot', 'themathqueen'] joelriou
assignee:joelriou
3-85994
3 days ago
10-61778
10 days ago
12-35158
12 days
31134 thorimur
author:thorimur
chore: use `whenLinterActivated` in linters Replaces boilerplate in linters with `whenLinterActivated` or `whenLinterOption` where possible. --- - [ ] depends on: #31133 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict 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 4 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] grunweg
assignee:grunweg
3-85963
3 days ago
unknown
unknown
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 - [x] depends on: #32719 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) brownian t-measure-probability 279/0 Mathlib.lean,Mathlib/Probability/Distributions/Gaussian/HasGaussianLaw/Basic.lean,Mathlib/Probability/Distributions/Gaussian/HasGaussianLaw/Def.lean 3 7 ['EtienneC30', 'RemyDegenne', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] kex-y
assignee:kex-y
3-71671
3 days ago
3-71073
3 days ago
37-74411
37 days
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) --- *This PR continues the work from #4197.* *Original PR: https://github.com/leanprover-community/mathlib4/pull/4197*
WIP t-category-theory large-import t-topology 36950/376 Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Free.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/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/ConnectShortExact.lean,Mathlib/Algebra/Homology/DerivedCategory/Basic.lean,Mathlib/Algebra/Homology/DerivedCategory/DerivabilityStructureInjectives.lean,Mathlib/Algebra/Homology/DerivedCategory/Fractions.lean,Mathlib/Algebra/Homology/DerivedCategory/FullyFaithful.lean,Mathlib/Algebra/Homology/DerivedCategory/HomologySequence.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/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/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/Acyclic.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/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/HomotopyFiber.lean,Mathlib/Algebra/Homology/LeftResolution/Basic.lean,Mathlib/Algebra/Homology/LeftResolution/CochainComplex.lean,Mathlib/Algebra/Homology/LeftResolution/CochainComplexMinus.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/Homology.lean,Mathlib/Algebra/Homology/ShortComplex/Images.lean,Mathlib/Algebra/Homology/ShortComplex/LeftHomology.lean,Mathlib/Algebra/Homology/ShortComplex/Preadditive.lean,Mathlib/Algebra/Homology/ShortComplex/Refinements.lean,Mathlib/Algebra/Homology/ShortComplex/RightHomology.lean,Mathlib/Algebra/Homology/ShortComplex/ShortComplexFive.lean,Mathlib/Algebra/Homology/ShortComplex/ShortComplexFour.lean,Mathlib/Algebra/Homology/ShortComplex/ULift.lean,Mathlib/Algebra/Homology/Single.lean,Mathlib/Algebra/Homology/SpectralObject/Basic.lean,Mathlib/Algebra/Homology/SpectralObject/Convergence.lean,Mathlib/Algebra/Homology/SpectralObject/Cycles.lean 280 4 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
3-70474
3 days ago
unknown
unknown
33690 Ljon4ik4
author:Ljon4ik4
feat: Defining Lie Rinehart algebras This PR provides the basics of Lie-Rinehart algebras: * Definition of the objects and homomorphism * Composition of LR-homomorphisms is a homomorphisms * Derivations of a commutative algebra are a Lie-Rinehart algebra * The anchor map of a Lie Rinehart algebra is a Lie Rinehart morphism Lie Rinehart algebras are an important structure: They naturally appear in the context of Lie algebroids and singular foliations in differential geometry. They also permit do define de-Rham type cohomology theories in all of these cases. We are working on more of the theory of Lie-Rinehart algebras with Sven Holtrop (@stholtrop). (Maybe it would make sense to have a mathlib branch for further developments?) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra new-contributor awaiting-author
label:t-algebra$
179/0 Mathlib.lean,Mathlib/Algebra/LieRinehartAlgebra/Defs.lean,Mathlib/RingTheory/Derivation/Lie.lean 3 18 ['Ljon4ik4', 'github-actions', 'kim-em'] nobody
3-64101
3 days ago
8-29712
8 days ago
0-5590
1 hour
33709 wangying11123
author:wangying11123
feat(Analysis/Convex/Between): Add wbtw_of_sameRay_vsub_left add wbtw_of_sameRay_vsub_left Main additions `wbtw_of_sameRay_vsub_left` if the vectors from a point x to points y and z lie on the same ray, then y is weakly between x and z, or z is weakly between x and y. new-contributor t-convex-geometry 24/0 Mathlib/Analysis/Convex/Between.lean 1 3 ['MichaelStollBayreuth', 'github-actions'] nobody
3-54771
3 days ago
7-80090
7 days ago
7-79910
7 days
33254 SnirBroshi
author:SnirBroshi
feat(Data/Nat/Lattice): `¬BddAbove s → sSup s = 0` --- Note that it can also be proven `by simp [h]` after the `ConditionallyCompleteLinearOrderBot` instance below it. The theorem name matches the same theorems for other types: `Int.csSup_of_not_bdd_above`, `Real.sSup_of_not_bddAbove`, `NNReal.sSup_of_not_bddAbove`. Also renamed related `Int` theorems to conform to the naming conventions. [Zulip](https://leanprover.zulipchat.com/#narrow/channel/217875-Is-there-code-for-X.3F/topic/.60.C2.ACBddAbove.20s.20.E2.86.92.20sSup.20s.20.3D.200.60/with/565275221) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data 15/4 Mathlib/Data/Int/ConditionallyCompleteOrder.lean,Mathlib/Data/Nat/Lattice.lean 2 3 ['SnirBroshi', 'artie2000', 'github-actions', 'vihdzp'] nobody
3-53715
3 days ago
21-50061
21 days ago
21-69497
21 days
32971 Paul-Lez
author:Paul-Lez
feat(Data/Finsupp/Pointwise): generalise pointwise scalar multiplication of finsupps This PR continues the work from #24050. Original PR: https://github.com/leanprover-community/mathlib4/pull/24050 t-data 7/4 Mathlib/Data/Finsupp/Pointwise.lean 1 3 ['Paul-Lez', 'artie2000', 'github-actions'] pechersky
assignee:pechersky
3-52676
3 days ago
29-59037
29 days ago
29-58857
29 days
32984 artie2000
author:artie2000
refactor: remove order instances from `SetLike` * Remove order instances from `SetLike` * Add class `IsConcreteLE` for `SetLike` instances whose map is order-preserving See discussion at https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Abstracting.20the.20substructure.20lattice.20construction/with/563952738 --- - [ ] depends on: #33801 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR t-data t-meta 375/146 Mathlib/Algebra/Algebra/NonUnitalSubalgebra.lean,Mathlib/Algebra/Algebra/Subalgebra/Basic.lean,Mathlib/Algebra/Field/Subfield/Defs.lean,Mathlib/Algebra/Group/Subgroup/Defs.lean,Mathlib/Algebra/Group/Submonoid/Defs.lean,Mathlib/Algebra/Group/Subsemigroup/Defs.lean,Mathlib/Algebra/Lie/Subalgebra.lean,Mathlib/Algebra/Lie/Submodule.lean,Mathlib/Algebra/Module/Submodule/Defs.lean,Mathlib/Algebra/Order/Group/Cone.lean,Mathlib/Algebra/Order/Group/Ideal.lean,Mathlib/Algebra/Order/Ring/Cone.lean,Mathlib/Algebra/Order/Ring/Ordering/Defs.lean,Mathlib/Algebra/Ring/Subring/Defs.lean,Mathlib/Algebra/Ring/Subsemiring/Defs.lean,Mathlib/Algebra/Star/NonUnitalSubalgebra.lean,Mathlib/Algebra/Star/Subalgebra.lean,Mathlib/Algebra/Star/Subsemiring.lean,Mathlib/AlgebraicGeometry/AffineScheme.lean,Mathlib/AlgebraicGeometry/Cover/Open.lean,Mathlib/AlgebraicGeometry/Limits.lean,Mathlib/AlgebraicGeometry/Morphisms/Basic.lean,Mathlib/AlgebraicGeometry/Morphisms/Separated.lean,Mathlib/AlgebraicGeometry/ProjectiveSpectrum/Basic.lean,Mathlib/AlgebraicGeometry/Scheme.lean,Mathlib/AlgebraicGeometry/StructureSheaf.lean,Mathlib/Analysis/Convex/Body.lean,Mathlib/Analysis/Convex/Cone/Basic.lean,Mathlib/Analysis/Convex/Cone/Dual.lean,Mathlib/Analysis/InnerProductSpace/Projection/FiniteDimensional.lean,Mathlib/Analysis/VonNeumannAlgebra/Basic.lean,Mathlib/CategoryTheory/Groupoid/Subgroupoid.lean,Mathlib/Combinatorics/SimpleGraph/Ends/Defs.lean,Mathlib/Combinatorics/Young/YoungDiagram.lean,Mathlib/Data/Finset/Defs.lean,Mathlib/Data/SetLike/Basic.lean,Mathlib/Data/Sym/Sym2.lean,Mathlib/FieldTheory/IntermediateField/Basic.lean,Mathlib/Geometry/Convex/Cone/Basic.lean,Mathlib/Geometry/Euclidean/Sphere/Power.lean,Mathlib/Geometry/Euclidean/Sphere/Tangent.lean,Mathlib/Geometry/Manifold/ChartedSpace.lean,Mathlib/Geometry/RingedSpace/Basic.lean,Mathlib/GroupTheory/GroupAction/SubMulAction.lean,Mathlib/GroupTheory/GroupAction/SubMulAction/Combination.lean,Mathlib/GroupTheory/Sylow.lean,Mathlib/LinearAlgebra/AffineSpace/AffineSubspace/Defs.lean,Mathlib/LinearAlgebra/Projectivization/Subspace.lean,Mathlib/ModelTheory/Definability.lean,Mathlib/ModelTheory/ElementarySubstructures.lean,Mathlib/ModelTheory/Substructures.lean,Mathlib/ModelTheory/Types.lean,Mathlib/NumberTheory/NumberField/FractionalIdeal.lean,Mathlib/Order/Atoms.lean,Mathlib/Order/BooleanSubalgebra.lean,Mathlib/Order/BourbakiWitt.lean,Mathlib/Order/Closure.lean,Mathlib/Order/CompleteSublattice.lean,Mathlib/Order/Ideal.lean,Mathlib/Order/PFilter.lean,Mathlib/Order/Partition/Basic.lean,Mathlib/Order/Preorder/Chain.lean,Mathlib/Order/Sublattice.lean,Mathlib/Order/Sublocale.lean,Mathlib/Order/UpperLower/CompleteLattice.lean,Mathlib/Order/UpperLower/Relative.lean,Mathlib/RepresentationTheory/Subrepresentation.lean,Mathlib/RingTheory/DedekindDomain/Different.lean,Mathlib/RingTheory/DedekindDomain/Factorization.lean,Mathlib/RingTheory/DedekindDomain/Ideal/Basic.lean,Mathlib/RingTheory/DividedPowers/SubDPIdeal.lean,Mathlib/RingTheory/FilteredAlgebra/Basic.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/RingTheory/GradedAlgebra/Homogeneous/Submodule.lean,Mathlib/RingTheory/GradedAlgebra/Homogeneous/Subsemiring.lean,Mathlib/RingTheory/NonUnitalSubring/Defs.lean,Mathlib/RingTheory/NonUnitalSubsemiring/Defs.lean,Mathlib/RingTheory/TwoSidedIdeal/Basic.lean,Mathlib/RingTheory/Valuation/ValuationSubring.lean,Mathlib/SetTheory/Descriptive/Tree.lean,Mathlib/SetTheory/ZFC/Basic.lean,Mathlib/Topology/Algebra/Group/ClosedSubgroup.lean,Mathlib/Topology/Algebra/Module/ClosedSubmodule.lean,Mathlib/Topology/Algebra/OpenSubgroup.lean,Mathlib/Topology/CWComplex/Classical/Basic.lean,Mathlib/Topology/Category/TopCat/OpenNhds.lean,Mathlib/Topology/Sets/Closeds.lean,Mathlib/Topology/Sets/Compacts.lean,Mathlib/Topology/Sets/Opens.lean,Mathlib/Topology/Sets/Order.lean,Mathlib/Topology/Sheaves/SheafCondition/Sites.lean,Mathlib/Topology/Sheaves/Stalks.lean,Mathlib/Topology/Spectral/Prespectral.lean,MathlibTest/FBinop.lean 98 31 ['Vierkantor', 'alreadydone', 'artie2000', 'github-actions', 'mathlib4-dependent-issues-bot'] nobody
3-51617
3 days ago
3-51618
3 days ago
2-802
2 days
32888 staroperator
author:staroperator
feat(Tactic/FunProp): make `fun_prop` able to tag `→` and `∀` by representing forall as a function application internally. Also tag `Measurable.imp` and `Measurable.forall` which were rejected by `fun_prop`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta 34/1 Mathlib/Lean/Expr/Basic.lean,Mathlib/MeasureTheory/MeasurableSpace/Constructions.lean,Mathlib/Tactic/FunProp/Mor.lean,MathlibTest/fun_prop.lean 4 12 ['JovanGerb', 'Komyyy', 'github-actions', 'staroperator'] eric-wieser
assignee:eric-wieser
3-45638
3 days ago
3-46369
3 days ago
11-74564
11 days
33336 fbarroero
author:fbarroero
feat(NumberTheory/MahlerMeasure): Kronecker's Theorem for the Mahler Measure This PR adds Kronecker's Theorem for the Mahler Measure, which characterizes integer polynomials with Mahler measure equal to 1. The key mathematical contribution is proving that such polynomials have all their nonzero complex roots as roots of unity, and consequently must be divisible by cyclotomic polynomials. Main result ``` Polynomial.pow_eq_one_of_mahlerMeasure_eq_one {p : ℤ[X]} (h : (map (castRingHom ℂ) p).mahlerMeasure = 1) {z : ℂ} (hz₀ : z ≠ 0) (hz : z ∈ p.aroots ℂ) : ∃ n, 0 < n ∧ z ^ n = 1 ``` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-number-theory 128/9 Mathlib/Algebra/Order/BigOperators/Ring/Multiset.lean,Mathlib/NumberTheory/MahlerMeasure.lean 2 25 ['MichaelStollBayreuth', 'copilot-pull-request-reviewer', 'github-actions', 'mathlib4-merge-conflict-bot'] tb65536
assignee:tb65536
3-43363
3 days ago
3-43363
3 days ago
11-12464
11 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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-euclidean-geometry 261/7 Mathlib/Geometry/Euclidean/Sphere/OrthRadius.lean,Mathlib/Geometry/Euclidean/Sphere/Tangent.lean 2 27 ['eric-wieser', 'github-actions', 'jsm28', 'mathlib4-dependent-issues-bot'] JovanGerb
assignee:JovanGerb
3-35459
3 days ago
10-54645
10 days ago
43-63808
43 days
33845 bjornsolheim
author:bjornsolheim
feat(Analysis/Convex): barycenter of a standard simplex barycenter of a standard simplex --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis 26/0 Mathlib/Analysis/Convex/StdSimplex.lean 1 5 ['bjornsolheim', 'eric-wieser', 'github-actions'] nobody
3-33332
3 days ago
3-31817
3 days ago
3-55344
3 days
33840 vihdzp
author:vihdzp
feat(SetTheory/Ordinal/CantorNormalForm): Evaluate a Finsupp as a CNF --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-set-theory 191/18 Mathlib/SetTheory/Ordinal/Arithmetic.lean,Mathlib/SetTheory/Ordinal/CantorNormalForm.lean 2 3 ['github-actions', 'plp127', 'vihdzp'] nobody
3-32713
3 days ago
3-31762
3 days ago
3-36650
3 days
33312 YuvalFilmus
author:YuvalFilmus
feat(Polynomial/Chebyshev): formulas for iterated derivatives of T and U at 1 The main results are `iterate_derivative_T_eval_one` and `iterate_derivative_U_eval_one`. These are derived using recurrences which for at every point, and in particular, `iterate_derivative_T_eval_zero` and `iterate_derivative_U_eval_zero` gives the recurrences at zero. In principle, by combining with #33311, one can compute the explicit formula for the derivative at zero. A subsequent PR will derive consequences for these polynomials over the reals (these should work for every field). The file is getting rather long — not sure what to do about it. --- - [ ] depends on: #33283 - [ ] depends on: #33306 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 110/0 Mathlib/RingTheory/Polynomial/Chebyshev.lean 1 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] Vierkantor
assignee:Vierkantor
3-31256
3 days ago
7-51576
7 days ago
7-52899
7 days
33714 idontgetoutmuch
author:idontgetoutmuch
Riemannian metrics exist II Supersedes https://github.com/leanprover-community/mathlib4/pull/33519 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-differential-geometry new-contributor 1269/0 Mathlib.lean,Mathlib/Geometry/Manifold/ExistsRiemannianMetricTangentSpace.lean,Mathlib/Geometry/Manifold/PartitionOfUnity.lean 3 3 ['github-actions', 'grunweg', 'idontgetoutmuch'] PatrickMassot
assignee:PatrickMassot
3-31254
3 days ago
6-85595
6 days ago
6-85415
6 days
33740 SnirBroshi
author:SnirBroshi
chore(Order/CompleteLattice/Basic): generalize many theorems to `CompleteSemilattice{Sup/Inf}` --- I believe some of these can be generalized further, this PR takes a small step. This might also allow half of these to be deleted thanks to `to_dual` somehow. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order 212/178 Mathlib/Order/CompleteLattice/Basic.lean,Mathlib/Order/Interval/Set/Disjoint.lean 2 8 ['JovanGerb', 'SnirBroshi', 'github-actions', 'vihdzp'] Vierkantor
assignee:Vierkantor
3-31253
3 days ago
6-71189
6 days ago
6-71009
6 days
33753 SnO2WMaN
author:SnO2WMaN
doc(1000.yaml): Mention Tarski's Undefinability Theorem in FFL --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor 3/0 docs/1000.yaml 1 3 ['SnO2WMaN', 'SnirBroshi', 'github-actions'] mariainesdff
assignee:mariainesdff
3-31249
3 days ago
4-84811
4 days ago
6-75113
6 days
33760 JovanGerb
author:JovanGerb
feat(Order/Bounds/Basic): use `to_dual` - part 1 This PR uses `to_dual` in the first half of `Order/Bounds/Basic`, and in `Order/Bounds/Defs`, and also tags `Iio`/`Ioi` and `Iic`/`Ici`. This dualization went quite smoothly. The lemma `HasSubset.Subset.iscofinalfor` has been renamed to use correct capitalization (so that the name can be translated automatically), and has been deprecated. A new definition defined in this PR is `IsCoinitial` as a dual to `IsCofinal`, because `IsCoinitialFor` already existed as a dual to `IsCofinalFor`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-order 127/282 Mathlib/Order/Bounds/Basic.lean,Mathlib/Order/Bounds/Defs.lean,Mathlib/Order/Interval/Set/Defs.lean,Mathlib/Tactic/Translate/ToDual.lean 4 4 ['JovanGerb', 'github-actions', 'vihdzp'] Vierkantor
assignee:Vierkantor
3-31247
3 days ago
4-19277
4 days ago
4-19097
4 days
33774 SnO2WMaN
author:SnO2WMaN
doc(100.yaml, 1000.yaml): Update about Gödel's Incompleteness Theorem --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor 4/4 docs/100.yaml,docs/1000.yaml 2 2 ['github-actions'] thorimur
assignee:thorimur
3-31243
3 days ago
4-85029
4 days ago
4-84849
4 days
33860 DavidLedvinka
author:DavidLedvinka
feat(Probability): Add Cauchy distribution t-measure-probability 125/0 Mathlib.lean,Mathlib/Probability/Distributions/Cauchy.lean 2 1 ['github-actions'] nobody
3-29734
3 days ago
3-28863
3 days ago
3-28683
3 days
33791 PhoenixIra
author:PhoenixIra
feat: Generalization of FixedPointApproximants to CompletePartialOrder --- This PR provides a generalization of FixedPointApproximants to CompletePartialOrder. Not every theorem can be generalized, as sometimes we require additional conditions (namely `x ≤ f x`) in order to guarantee that the set is directed and thus the supremum is well-defined. This is not necessary in a CompleteLattice. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor 255/42 Mathlib/Order/CompletePartialOrder.lean,Mathlib/SetTheory/Ordinal/FixedPointApproximants.lean 2 7 ['github-actions', 'vihdzp'] vihdzp
assignee:vihdzp
3-29241
3 days ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR t-euclidean-geometry 419/7 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-25993
3 days ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR t-euclidean-geometry 478/9 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-25970
3 days ago
unknown
unknown
33852 zcyemi
author:zcyemi
feat(LinearAlgebra/AffineSpace/Independent): Add affineCombination_eq_lineMap_iff_weight_lineMap --- ```lean theorem AffineIndependent.affineCombination_eq_lineMap_iff_weight_lineMap {p : ι → P} (ha : AffineIndependent k p) {w w₁ w₂ : ι → k} {s : Finset ι} (hw : ∑ i ∈ s, w i = 1) (hw₁ : ∑ i ∈ s, w₁ i = 1) (hw₂ : ∑ i ∈ s, w₂ i = 1) (c : k) : s.affineCombination k p w = AffineMap.lineMap (s.affineCombination k p w₁) (s.affineCombination k p w₂) c ↔ ∀ i ∈ s, w i = AffineMap.lineMap (w₁ i) (w₂ i) c := by ``` This theorem is a parameterized reformulation of `affineCombination_mem_affineSpan_pair`. It is convenient for rewriting when a concrete `lineMap` parameter is given. t-algebra
label:t-algebra$
23/0 Mathlib/LinearAlgebra/AffineSpace/Independent.lean 1 4 ['github-actions', 'jsm28', 'zcyemi'] nobody
3-25951
3 days ago
3-24254
3 days ago
3-30373
3 days
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-euclidean-geometry blocked-by-other-PR 578/9 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 5 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
3-25931
3 days ago
53-27787
53 days ago
0-583
9 minutes
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) IMO blocked-by-other-PR 2459/65 Archive.lean,Archive/Imo/Imo2024Q4.lean,Mathlib.lean,Mathlib/Analysis/Convex/Side.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,Mathlib/Geometry/Euclidean/Sphere/OrthRadius.lean,Mathlib/Geometry/Euclidean/Sphere/PolePolar.lean,Mathlib/Geometry/Euclidean/Sphere/Tangent.lean 13 5 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
3-25914
3 days ago
unknown
unknown
27702 FLDutchmann
author:FLDutchmann
feat(NumberTheory/SelbergSieve): define Lambda-squared sieves and prove important properties This PR continues the work from #22052. Original PR: https://github.com/leanprover-community/mathlib4/pull/22052 - [x] depends on: #27820 t-number-theory delegated 186/7 Mathlib/NumberTheory/SelbergSieve.lean 1 42 ['FLDutchmann', 'MichaelStollBayreuth', 'bryangingechen', 'github-actions', 'jcommelin', 'mathlib-bors', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] MichaelStollBayreuth
assignee:MichaelStollBayreuth
3-23622
3 days ago
35-7337
35 days ago
15-79295
15 days
33697 artie2000
author:artie2000
feat(FieldTheory): real closed field * Define real closed fields * Prove some very basic properties --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
117/0 Mathlib.lean,Mathlib/FieldTheory/IsRealClosed/Basic.lean 2 40 ['artie2000', 'github-actions', 'vihdzp'] dagurtomas
assignee:dagurtomas
3-23588
3 days ago
3-51404
3 days ago
7-79671
7 days
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 --- t-ring-theory 203/0 Mathlib.lean,Mathlib/LinearAlgebra/Finsupp/LinearCombination.lean,Mathlib/RingTheory/SimpleRing/TensorProduct.lean,Mathlib/RingTheory/TwoSidedIdeal/Operations.lean 4 50 ['Ruben-VandeVelde', 'Whysoserioushah', 'eric-wieser', 'github-actions', 'kbuzzard', 'kckennylau', 'mathlib4-merge-conflict-bot', 'vlad902'] kbuzzard
assignee:kbuzzard
3-22489
3 days ago
4-1221
4 days ago
10-57027
10 days
13158 erdOne
author:erdOne
refactor(RingTheory/OreLocalization/Module): remove `LocalizedModule.mk`. --- - [x] depends on: #13151 - [ ] depends on: #13156 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra blocked-by-other-PR
label:t-algebra$
49/48 Mathlib/RingTheory/OreLocalization/Basic.lean,Mathlib/RingTheory/OreLocalization/Module.lean 2 2 ['leanprover-community-mathlib4-bot', 'urkud'] nobody
3-19692
3 days ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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 12 ['YaelDillies', 'adomani', 'github-actions', 'grunweg', 'jcommelin', 'urkud'] nobody
3-19599
3 days ago
unknown
unknown
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). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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 8 ['github-actions', 'grunweg', 'kbuzzard', 'mathlib4-merge-conflict-bot', 'urkud'] nobody
3-19476
3 days ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author CI merge-conflict 1/1 bors.toml 1 5 ['bryangingechen', 'eric-wieser', 'github-actions', 'mathlib4-merge-conflict-bot', 'urkud'] nobody
3-19388
3 days ago
75-55184
75 days ago
0-64037
17 hours
33863 urkud
author:urkud
feat: generalize some lemmas about LTOs Currently, lemmas about `Filter.map ((↑) : Set.Iio a → X) Filter.atTop` etc assume that the ambient type is densely ordered. However, it suffices to require that `a` is an `Order.IsSuccPrelimit`. Make this generalization and move the lemmas to a new file. Also, use the new lemmas to drop a `[DenselyOrdered _]` assumption in one lemma in measure theory. These more precise statements are also useful when dealing with, e.g., LTOs defined by ordinals. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 226/130 Mathlib.lean,Mathlib/Analysis/SpecialFunctions/Exp.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Arctan.lean,Mathlib/MeasureTheory/Measure/Hausdorff.lean,Mathlib/MeasureTheory/Measure/MeasureSpace.lean,Mathlib/Topology/Order/AtTopBotIxx.lean,Mathlib/Topology/Order/DenselyOrdered.lean 7 1 ['github-actions'] nobody
3-17890
3 days ago
3-16171
3 days ago
3-15991
3 days
33105 Timeroot
author:Timeroot
feat(BoundedOrder): add `finiteness` rule for ite and dite The `finiteness` tactic could do well to recurse on if statements by trying to prove both branches are finite; this adds the appropriate theorem. In principal this theorem could go even a bit higher in the import hierarchy, but this means importing the finiteness attribute even earlier, the finiteness tactic cannot be used that early, and I fail to imagine why someone would want this theorem /except/ for the finiteness tactic really. (Normally one can just `split`.) Upstreamed from [quantumInfo](https://github.com/Timeroot/Lean-QuantumInfo) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order awaiting-author t-meta 31/2 Mathlib/MeasureTheory/Constructions/ProjectiveFamilyContent.lean,Mathlib/Order/BoundedOrder/Basic.lean,Mathlib/Tactic/Finiteness.lean,MathlibTest/finiteness.lean 4 7 ['Timeroot', 'github-actions', 'grunweg', 'leanprover-radar'] grunweg
assignee:grunweg
3-17152
3 days ago
unknown
unknown
32440 thorimur
author:thorimur
feat: make the `unusedDecidableInType` linter fire when `Decidable*` instances are used only inside of proofs in the type This PR adjusts the `unusedDecidableInType` to prevent false negatives on declarations that only use `Decidable*` hypotheses in proofs that appear in the type. That is, the linter now fires when the `Decidable*` linter is unused outside of proofs. This PR also changes the warning message to be more direct, and indicates when the instance appears only in a proof (vs. not appearing at all). We exempt some deprecated lemmas in `Mathlib.Analysis.Order.Matrix` which the linter now fires on. (Presumably, most prior violations had been cleaned up by #10235, which also detected such lemmas.) Note that this took some tinkering to achieve sufficient performance. We use the following novel(?) "dolorous telescope" strategy (so named due to introducing `sorry`s) to avoid traversing the whole type: - when encountering an instance binder of concern, telescope to create an fvar. - when encountering any other binder, instantiate it with `sorry`. - as we proceed, collect the free variables from these expressions which do not appear in proofs. Since the instances of concern are the only free variables, free variable collection avoids traversing many subexpressions by checking for `hasFVar`, which is a computed field accessible in constant time. Perhaps surprisingly, this is (on net) more performant than using `eraseProofs` and then detecting dependence via bvars. We also implement an `Expr`-level early exit for most types by checking if they bind any instance of concern first. (This adds a very small overhead to types which *do* have an instance of concern, but the check is very fast.) This also adds a profiler category to this linter. Note: we still have yet to optimize (pre)-infotree traversal performance, and have yet to avoid proofs that appear in the value of definitions. However, this PR sets us up to do so. --- ## Notes on performance You might be wondering if this *is* actually a faster strategy, seeing as the bench is quite noisy. To determine this, I made a copy of the linter which I could vary without rebuilding mathlib, and profiled the relevant component locally on all imported declarations in Mathlib by linting the `eoi` token: ```lean module public meta import Lean public import Mathlib.Tactic.Linter.UnusedInstancesInTypeCopy import all Mathlib.Tactic.Linter.UnusedInstancesInTypeCopy open Lean Meta Elab Term Command Mathlib.Linter.UnusedInstancesInType meta section local instance : Insert Name NameSet where insert := fun n s => s.insert n def runCopy : Linter where run stx := do if stx.isOfKind ``Parser.Command.eoi then let opts := (← getOptions).setBool `profiler true let consts := (← getEnv).constants.map₁ -- The following expose private decls in their types, so break `MetaM` methods: let badRecs : NameSet := {`IO.Promise.casesOn, `IO.Promise.recOn, `IO.Promise.rec} profileitM Exception "control" opts do for (n,_) in consts do liftTermElabM do unless n.isInternalDetail || badRecs.contains n do pure () profileitM Exception "bench" opts do for (n,cinfo) in consts do unless n.isInternalDetail || badRecs.contains n do cinfo.toConstantVal.onUnusedInstancesInTypeWhere isDecidableVariant fun _ _ => pure () initialize addLinter runCopy ``` (This could have been done in a `run_cmd`, but I wanted to replicate the circumstances of linting as closely as possible, just in case it introduced mysterious async effects.) Then, in a separate file, I imported `Mathlib` and the above linter, and cycled through reading out the result and editing the underlying component then rebuilding. The control was reliably ~1.07-1.12s. The different strategies came out as follows (the following values are not averaged, but are representative): | | without early exit | with early exit | | ---: | :---: | :---: | | `eraseProofs` | 97.4s | 6.82s | | dolorous telescope | 20.3s | 3.99s | As you can see, the early exit cuts the absolute value (and therefore the absolute difference) down dramatically. But seeing as this lays the groundwork for linting defs and will be used for more linters (with wider scopes, and less early exit opportunities), I think we should opt for the more performant version even though there's some extra complexity. :) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-linter 199/51 Mathlib/Analysis/Matrix/Order.lean,Mathlib/Lean/Expr/Basic.lean,Mathlib/Tactic/Linter/UnusedInstancesInType.lean,MathlibTest/UnusedInstancesInType.lean 4 30 ['github-actions', 'grunweg', 'leanprover-radar', 'mathlib4-merge-conflict-bot', 'thorimur'] joneugster
assignee:joneugster
3-13225
3 days ago
4-53753
4 days ago
32-74827
32 days
32892 Parcly-Taxel
author:Parcly-Taxel
feat(Analysis/SpecialFunctions): arithmetic-geometric mean t-analysis 211/0 Mathlib.lean,Mathlib/Analysis/SpecialFunctions/AGM.lean 2 10 ['AntoineChambert-Loir', 'Parcly-Taxel', 'github-actions', 'j-loreaux'] sgouezel
assignee:sgouezel
3-12702
3 days ago
22-43648
22 days ago
8-45222
8 days
33832 alreadydone
author:alreadydone
feat(Algebra): localization preserves unique factorization --- - [ ] depends on: #33851 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR t-algebra bench-after-CI
label:t-algebra$
159/16 Mathlib/Algebra/BigOperators/Group/Finset/Basic.lean,Mathlib/Algebra/GroupWithZero/Associated.lean,Mathlib/Algebra/Ring/Regular.lean,Mathlib/GroupTheory/MonoidLocalization/Basic.lean,Mathlib/GroupTheory/MonoidLocalization/MonoidWithZero.lean,Mathlib/GroupTheory/MonoidLocalization/UniqueFactorization.lean,Mathlib/RingTheory/Localization/Defs.lean 7 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
3-977
3 days ago
unknown
unknown
31706 Thmoas-Guan
author:Thmoas-Guan
feat(Algebra/ModuleCat): `ModuleCat.uliftFunctor` Add `ModuleCat.uliftFunctor` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra awaiting-author maintainer-merge
label:t-algebra$
108/0 Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Ulift.lean 2 20 ['Thmoas-Guan', 'dagurtomas', 'erdOne', 'github-actions', 'mathlib4-merge-conflict-bot', 'robin-carlier'] mattrobball
assignee:mattrobball
2-81991
2 days ago
2-81991
2 days ago
14-79739
14 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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology 257/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,docs/references.bib 7 6 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'robin-carlier'] ADedecker
assignee:ADedecker
2-79271
2 days ago
2-77050
2 days ago
54-79848
54 days
33872 WenrongZou
author:WenrongZou
feat(RingTheory/MvPowerSeries): some inequalities related to order Some inequalities related to order of (mv) power series. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-ring-theory 82/9 Mathlib/RingTheory/MvPowerSeries/Order.lean,Mathlib/RingTheory/PowerSeries/Order.lean,Mathlib/RingTheory/PowerSeries/Substitution.lean 3 1 ['github-actions'] nobody
2-78492
2 days ago
unknown
unknown
33764 IvanRenison
author:IvanRenison
feat(Combinatorics/SimpleGraph/Diam): drop `Finite α` from `ediam_le_two_mul_radius` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics 22/5 Mathlib/Combinatorics/SimpleGraph/Diam.lean 1 3 ['Rida-Hamadani', 'github-actions', 'vlad902'] nobody
2-78344
2 days ago
3-67777
3 days ago
6-53746
6 days
31595 astrainfinita
author:astrainfinita
chore: redefine `Ideal.IsPrime` Redefine `Ideal.IsPrime` to make it correct for non-commutative cases --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict
label:t-algebra$
330/100 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/Ideal/Quotient/Operations.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 22 29 ['alreadydone', 'artie2000', 'astrainfinita', 'erdOne', 'github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'mathlib4-merge-conflict-bot'] alreadydone
assignee:alreadydone
2-76800
2 days ago
4-48894
4 days ago
28-50719
28 days
32974 jano-wol
author:jano-wol
feat: golf eq_top_of_invtSubmodule_ne_bot --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) delegated t-algebra
label:t-algebra$
111/161 Mathlib/Algebra/Lie/Weights/IsSimple.lean,Mathlib/Algebra/Lie/Weights/Killing.lean,Mathlib/LinearAlgebra/RootSystem/Irreducible.lean 3 10 ['github-actions', 'jano-wol', 'mathlib-bors', 'mathlib4-merge-conflict-bot', 'ocfnash'] ocfnash
assignee:ocfnash
2-76577
2 days ago
2-76577
2 days ago
3-59216
3 days
33478 anishrajeev
author:anishrajeev
feat(ModelTheory): define a subset of the topology over complete types Define a subset of the Stone Space over a language expanded with countably many constants. Define the proposition to indicate if a language is countable. The subset's density and openness is a future goal to prove (have a branch where it is almost finished), in pursuit of formalizing the proof of the Omitting Types Theorem via properties of Baire spaces. - [ ] depends on: #32215 - [ ] depends on: #32546 t-logic blocked-by-other-PR new-contributor 160/1 Mathlib.lean,Mathlib/ModelTheory/Topology/Types.lean,Mathlib/ModelTheory/Types.lean,Mathlib/Tactic/Linter/DirectoryDependency.lean 4 7 ['NoneMore', 'anishrajeev', 'github-actions', 'mathlib4-dependent-issues-bot', 'tb65536'] nobody
2-73984
2 days ago
2-73985
2 days ago
10-30503
10 days
33874 joelriou
author:joelriou
feat(Algebra/Homology/ShortComplex): cycles can be computed with a limit kernel fork We make a few additions to the homology API, as it shall be necessary to formalize spectral sequences #33842. Let `S` be a short complex. The data of a kernel fork of `S.g` allows to compute `S.cycles`. Similarly, the data of a cokernel cofork of `S.f` allows to compute `S.opcycles`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-category-theory
label:t-algebra$
82/1 Mathlib/Algebra/Homology/ShortComplex/Basic.lean,Mathlib/Algebra/Homology/ShortComplex/Exact.lean,Mathlib/Algebra/Homology/ShortComplex/Homology.lean,Mathlib/Algebra/Homology/ShortComplex/LeftHomology.lean,Mathlib/Algebra/Homology/ShortComplex/RightHomology.lean 5 1 ['github-actions'] nobody
2-72706
2 days ago
unknown
unknown
26884 alreadydone
author:alreadydone
Universal cover TODO: construct locally constant predicate from a functor from the fundamental groupoid of a loc path connected, semilocally simply connected space to Type, and the associated covering space (as an etale space) --- - [x] depends on: #24983 - [x] depends on: #22771 - [ ] depends on: #31925 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-topology blocked-by-other-PR 900/165 Mathlib.lean,Mathlib/AlgebraicGeometry/Modules/Tilde.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 11 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
2-72377
2 days ago
unknown
unknown
33595 JovanGerb
author:JovanGerb
chore: remove some `backward.proofsInPublic` This PR removes some uses of `backward.proofsInPublic`. Most of these could be removed without any modification. In two of these I filled in some metavariables to the right value. The remaining cases also all complain about some metavariables being uninstantiated. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 4/21 Mathlib/Algebra/Group/End.lean,Mathlib/Algebra/Group/Equiv/Defs.lean,Mathlib/Algebra/Group/InjSurj.lean,Mathlib/Algebra/Group/Subgroup/Map.lean,Mathlib/Algebra/Group/Units/Hom.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Affine/Point.lean,Mathlib/Condensed/Discrete/Colimit.lean,Mathlib/Data/Finset/NoncommProd.lean,Mathlib/GroupTheory/Exponent.lean,Mathlib/GroupTheory/GroupAction/SubMulAction/OfFixingSubgroup.lean,Mathlib/GroupTheory/OreLocalization/Basic.lean,Mathlib/RingTheory/Extension/Cotangent/Basic.lean 12 2 ['github-actions', 'jcommelin'] nobody
2-71634
2 days ago
unknown
unknown
33879 joelriou
author:joelriou
feat(CategoryTheory/ComposableArrows): isIso_iff We introduce lemmas characterizing isomorphisms in `ComposableArrows C n` for small numbers `n`. We add autoparams (`by cat_disch`) for certain parameters. We also make definitions like `mk₂` reducible (instead of using the `simp` attribute), as it will allow to have `mk₂` in the LHS/RHS of simp lemmas in the formalization of spectral sequences #33842. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory 76/31 Mathlib/CategoryTheory/ComposableArrows/Basic.lean,Mathlib/CategoryTheory/ComposableArrows/Two.lean 2 1 ['github-actions'] nobody
2-71097
2 days ago
unknown
unknown
33437 joelriou
author:joelriou
feat(Algebra/Homology): short exact sequences with four terms The main definition in this file is `ComposableArrows.Exact.cokerIsoKer`: given an exact sequence `S` (involving at least four objects), this is the isomorphism from the cokernel of `S.map' k (k + 1)` to the kernel of `S.map' (k + 2) (k + 3)`. This will be used in the formalization of spectral sequences #33842. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-category-theory
label:t-algebra$
235/0 Mathlib.lean,Mathlib/Algebra/Homology/ExactSequence.lean,Mathlib/Algebra/Homology/ExactSequenceFour.lean 3 1 ['github-actions'] nobody
2-69901
2 days ago
unknown
unknown
33881 joelriou
author:joelriou
feat(CategoryTheory/ComposableArrows): API for the composition of four arrows This shall be used in the formalization of spectral sequences #33842. --- - [ ] depends on: #33879 - [ ] depends on: #33880 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory WIP blocked-by-other-PR 358/31 Mathlib.lean,Mathlib/CategoryTheory/ComposableArrows/Basic.lean,Mathlib/CategoryTheory/ComposableArrows/Four.lean,Mathlib/CategoryTheory/ComposableArrows/Three.lean,Mathlib/CategoryTheory/ComposableArrows/Two.lean 5 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
2-69559
2 days ago
unknown
unknown
33880 joelriou
author:joelriou
feat(CategoryTheory/ComposableArrows): API for the composition of three arrows This shall be used in the formalization of spectral sequences #33842. --- - [ ] depends on: #33879 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory WIP blocked-by-other-PR 197/31 Mathlib.lean,Mathlib/CategoryTheory/ComposableArrows/Basic.lean,Mathlib/CategoryTheory/ComposableArrows/Three.lean,Mathlib/CategoryTheory/ComposableArrows/Two.lean 4 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
2-69557
2 days ago
unknown
unknown
33875 joelriou
author:joelriou
feat(Algebra/Homology): an homology data from an epi-mono factorization Let `S` be a short complex in an abelian category. If `K` is a kernel of `S.g` and `Q` a cokernel of `S.f`, and `K ⟶ H ⟶ Q` is an epi-mono factorization of `K ⟶ S.X₂ ⟶ Q`, then `H` identifies to the homology of `S`. (That shall be used when computing the homology of the differentials on pages of spectral sequences #33842.) --- - [ ] depends on: #33874 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import WIP blocked-by-other-PR 255/5 Mathlib/Algebra/Homology/ShortComplex/Abelian.lean,Mathlib/Algebra/Homology/ShortComplex/Basic.lean,Mathlib/Algebra/Homology/ShortComplex/Exact.lean,Mathlib/Algebra/Homology/ShortComplex/Homology.lean,Mathlib/Algebra/Homology/ShortComplex/LeftHomology.lean,Mathlib/Algebra/Homology/ShortComplex/RightHomology.lean,Mathlib/CategoryTheory/Limits/Shapes/Equalizers.lean 7 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
2-69555
2 days ago
unknown
unknown
33883 joelriou
author:joelriou
feat(CategoryTheory/ObjectProperty): various additions This PR adds a few basic results about `ObjectProperty` that will be used in the formalization of spectral sequences #33842. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory 49/3 Mathlib/CategoryTheory/Limits/Shapes/ZeroObjects.lean,Mathlib/CategoryTheory/ObjectProperty/ContainsZero.lean,Mathlib/CategoryTheory/ObjectProperty/FullSubcategory.lean,Mathlib/CategoryTheory/ObjectProperty/Shift.lean 4 1 ['github-actions'] nobody
2-69526
2 days ago
2-62678
2 days ago
2-62498
2 days
32039 HugLycan
author:HugLycan
feat(Tactic/Positivity): handle non-zeroness in non-orders --- WIP... [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP new-contributor t-meta merge-conflict 528/131 Mathlib/Tactic/Positivity/Basic.lean,Mathlib/Tactic/Positivity/Core.lean,Mathlib/Tactic/Positivity/test_Basic.lean 3 3 ['github-actions', 'mathlib4-merge-conflict-bot'] nobody
2-69064
2 days ago
unknown
unknown
27557 chrisflav
author:chrisflav
feat(RingTheory/KrullDimension): generalize some results about local rings We generalize `ringKrullDim_le_ringKrullDim_add_card` to non-local rings by assuming `s ⊆ Ring.jacobson R` instead of `s ⊆ maximalIdeal R`. For this we show that if `R` is a Noetherian ring and `I` is an ideal contained in a prime ideal `p`, then the height of `p` is bounded by the sum of the height of the image of `p` in `R / I` and the span rank of `I`. --- - [x] depends on: #27538 - [x] depends on: #27510 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-ring-theory 125/44 Mathlib/RingTheory/Ideal/KrullsHeightTheorem.lean,Mathlib/RingTheory/Ideal/MinimalPrime/Basic.lean,Mathlib/RingTheory/Jacobson/Radical.lean,Mathlib/RingTheory/KrullDimension/Regular.lean 4 4 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
2-68249
2 days ago
4-80481
4 days ago
1-13214
1 day
33088 joelriou
author:joelriou
feat(AlgebraicTopology/ModelCategory): the left derivability structure We show that the inclusion of the full subcategory of cofibrant objects in a model category gives a left derivability structure (with respect to weak equivalences). --- - [x] depends on: #33084 - [x] depends on: #33085 - [x] depends on: #33086 - [ ] depends on: #33087 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebraic-topology t-category-theory WIP blocked-by-other-PR 392/0 Mathlib.lean,Mathlib/AlgebraicTopology/ModelCategory/CofibrantObjectHomotopy.lean,Mathlib/AlgebraicTopology/ModelCategory/DerivabilityStructureCofibrant.lean 3 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
2-68142
2 days ago
unknown
unknown
33233 jazzits
author:jazzits
feat(GroupTheory): add chosen group presentations and finitely presented groups This PR adds "chosen" generating systems and presentations of a group, and uses it to define and develop very basic notions around finitely presented groups in a way that integrates with `Mathlib.GroupTheory.PresentedGroup`. Main additions: * New file `Mathlib/GroupTheory/Presentation.lean`: - `Group.GeneratingSystem` and `Group.Presentation` (with kernel = normal closure hypothesis) - the canonical map `Presentation.toGroup` - an isomorphism `Presentation.equivPresentedGroup : PresentedGroup P.rels ≃* G` - transport of presentations along a group isomorphism (`Presentation.mapMulEquiv`) * New file `Mathlib/GroupTheory/FinitelyPresented.lean`: - `Group.FinitelyPresented` defined as existence of a finite presentation - equivalence `FinitelyPresented ↔ ∃ rels, PresentedGroup rels ≃* G` with finiteness hypotheses - canonical presentation of `PresentedGroup rels` - finitely presented groups are finitely generated The development is designed to reuse the existing `PresentedGroup` construction and avoids introducing a new quotient model for presented groups. No existing definitions are modified t-group-theory new-contributor awaiting-author 442/0 Mathlib.lean,Mathlib/GroupTheory/FinitelyPresented.lean,Mathlib/GroupTheory/Presentation.lean 3 13 ['github-actions', 'homeowmorphism', 'jazzits', 'kbuzzard', 'plp127', 'tb65536'] tb65536
assignee:tb65536
2-67915
2 days ago
unknown
unknown
33822 robin-carlier
author:robin-carlier
feat(Meta/CategoryTheory): `cancelIso` simproc In this PR, we define a `cancelIso` simplification procedure. The scope of the procedure is to recognize compositions of the form `f ≫ g` or `f ≫ g ≫ h` where `g` is inverse to `f`, and cancel them accordingly. This is particularly useful as more often than not, simp normal forms for isomorphisms do not easily make inverse pairs recognizable: `F.map (G.map (H.map e.hom))) ≫ F.map (G.map (H.map e.inv)))` is an expression in `simp`normal form, but using `Iso.hom_inv_id` requires backwards rewriting of `Functor.map_comp`. Because of this, many _ad hoc_ lemmas handling this pattern were added to the library, e.g `CategoryTheory.Iso.inv_hom_id_app_app_app`, `CategoryTheory.MonoidalCategory.hom_inv_whiskerRight`, etc. This simproc is an attempt at lessening the need for new extra lemmas of this form. The core working of the simproc is as follows: 1. When encountering a composition `f ≫ g`, check if the target of `g` is the source of `f` 2. If so, Try to synth an `IsIso` instance on `f` (In all the patterns mentioned above, such instances are available). Do nothing and return if there is no such instance. 4. Run `push inv` on both `inv f` and `g`, putting them in "inv-normal form" and compare the results. If they match, build (using the proofs provided by `push`) a proof of `f ≫ g = 𝟙 _`, and return it as the result of the procedure. In practice, the case where `g` itself is a composition is handled on its own, allowing the simproc to correctly fire on right-associated expressions (which are the chosen simp normal forms in category theory). Because this simproc relies on `push`, it is naturally extentable by means of rigorous `@[push]` annotations within the library. :robot: tests were initially generated by Gemini. --- While the particular problem that this simproc solves might intersect with the capabilities of grind, I believe it is an useful thing to have. In my experience, the place where its absence is most annoying is when carrying computation heavy proofs in bicategory theory, where I’ve encountered terms of the form `A ◁ B ◁ C ◁ D ◁ e.inv ▷ E ▷ F ▷ G ▷ H ≫ A ◁ B ◁ C ◁ D ◁ e.hom ▷ E ▷ F ▷ G ▷ H `, where `A, B, C' etc might have long names. Doing `show ... = 𝟙 _ by grind` would be very long. This has also value for goals is not currently solving due to lack of annotations, but whose simp normal forms make such terms appear. In the future, I think the infrastructure under this simproc might give a nice backend towards a cleaner implementation of the `rotate_iso%` elaborator I proposed in #25747, making it natively extendable via `@[push]` annotations. I am not very well versed in metaprogramming, so the main questions I would ask are - Is the `withReducible` useful? I put it as a safe measure to avoid triggering expensive def-eq checks, but I don’t know wether or not being in the `SimpM` monad wraps things with this transparency already? - Is the file in the right place? Should it be in the folder with other Simprocs despite being specialized to category theory? - I did not make it as a simproc that should fire by default, as I am slightly wary of the performances here, but maybe I’m overthinking it? - [x] depends on: #33820 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-category-theory t-meta merge-conflict 280/34 Mathlib.lean,Mathlib/AlgebraicTopology/SimplicialNerve.lean,Mathlib/CategoryTheory/Bicategory/Basic.lean,Mathlib/CategoryTheory/Category/Basic.lean,Mathlib/CategoryTheory/Comma/Basic.lean,Mathlib/CategoryTheory/Iso.lean,Mathlib/CategoryTheory/Limits/Shapes/Pullback/Categorical/Basic.lean,Mathlib/CategoryTheory/Monoidal/Category.lean,Mathlib/CategoryTheory/Monoidal/Closed/FunctorCategory/Groupoid.lean,Mathlib/CategoryTheory/NatIso.lean,Mathlib/CategoryTheory/Opposites.lean,Mathlib/Tactic.lean,Mathlib/Tactic/CategoryTheory/CancelIso.lean,MathlibTest/CategoryTheory/CancelIso.lean 14 54 ['JovanGerb', 'github-actions', 'leanprover-radar', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'plp127', 'robin-carlier'] nobody
2-67889
2 days ago
3-49972
3 days ago
0-13314
3 hours
33387 AntoineChambert-Loir
author:AntoineChambert-Loir
chore(LinearAlgebra/Transvection/Basic): mv Transvection.lean file to Transvection.Basic.lean In preparation for a long file about Dieudonné's theorem on the generation of the general and special linear groups, mv file#Mathlib/LinearAlgebra/Transvection.lean to file#Mathlib/LinearAlgebra/Transvection/Basic.lean --- - [ ] depends on: #33348 - [ ] depends on: #33347 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) file-removed t-algebra blocked-by-other-PR
label:t-algebra$
617/222 Mathlib.lean,Mathlib/LinearAlgebra/Determinant.lean,Mathlib/LinearAlgebra/Transvection.lean,Mathlib/LinearAlgebra/Transvection/Basic.lean 4 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
2-66851
2 days ago
unknown
unknown
33392 AntoineChambert-Loir
author:AntoineChambert-Loir
feat(LinearAlgebra/Transvection/Generation): non-exceptional case in Dieudonné's theorem We prove the theorem of [Dieudonné-1955][J. Dieudonné, “Sur les générateurs des groupes classiques”]. Let `K` be a division ring and `V` be a `K`-module. * `LinearEquiv.mem_transvections_pow_mul_dilatransvections_of_fixedReduce_eq_one`: If `e.fixedReduce = 1`, then `e` can be written as the product of `finrank K (V ⧸ e.fixedSubmodule) - 1` transvections and one dilatransvection. This is the first part of the non-exceptional case in Dieudonné's theorem. (This statement is not interesting when `e = 1`.) * `LinearEquiv.mem_transvections_pow_mul_dilatransvections_of_fixedReduce_ne_smul_id`: If `e.fixedReduce` is not a homothety, then `e` can be written as the product of `finrank K (V ⧸ e.fixedSubmodule) - 1` transvections and one dilatransvection. This is the second part of the non-exceptional case in Dieudonné's theorem. * `LinearEquiv.IsExceptional`: A linear equivalence `e : V ≃ₗ[K] V` is exceptional if `1 < finrank K (V ⧸ e.fixedSubmodule)` and if `e.fixedReduce` is a nontrivial homothety. * `LinearEquiv.mem_dilatransvections_pow_of_notIsExceptional`: This is the non-exceptional case in Dieudonné's theorem, as a combination of the two preceding statements. --- - [ ] depends on: #33348 - [ ] depends on: #33347 - [ ] depends on: #33387 - [ ] depends on: #33282 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra blocked-by-other-PR file-removed
label:t-algebra$
1412/222 Mathlib.lean,Mathlib/LinearAlgebra/Center.lean,Mathlib/LinearAlgebra/Determinant.lean,Mathlib/LinearAlgebra/FiniteDimensional/Lemmas.lean,Mathlib/LinearAlgebra/LinearIndependent/Lemmas.lean,Mathlib/LinearAlgebra/Transvection.lean,Mathlib/LinearAlgebra/Transvection/Basic.lean,Mathlib/LinearAlgebra/Transvection/Generation.lean 8 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
2-66544
2 days ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR t-differential-geometry 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
2-66483
2 days ago
unknown
unknown
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.) --- Needs some clean-up in both the immersions file, and need to move the helper results about embeddings to the correct location. - [x] depends on: #28793 - [ ] depends on: #28796 - [x] depends on: #28853 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR t-differential-geometry 331/15 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/Geometry/Manifold/SmoothEmbedding.lean 7 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
2-66473
2 days ago
unknown
unknown
25822 ScottCarnahan
author:ScottCarnahan
WIP: experiments with vertex algebras This is a testbed for various attempts at things. Please don't bother reviewing. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) --- *This PR continues the work from #25821.* *Original PR: https://github.com/leanprover-community/mathlib4/pull/25821* WIP large-import merge-conflict 8182/284 Mathlib.lean,Mathlib/Algebra/Lie/BaseChange.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/Lattice.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 42 25 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-merge-conflict-bot'] nobody
2-66290
2 days ago
unknown
unknown
33303 sinhp
author:sinhp
feat(CategoryTheory): The monads and comonads of locally cartesian closed categories --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-category-theory 405/8 Mathlib/CategoryTheory/Comma/Over/Basic.lean,Mathlib/CategoryTheory/LocallyCartesianClosed/ChosenPullbacksAlong.lean,Mathlib/CategoryTheory/LocallyCartesianClosed/Monad.lean 3 2 ['github-actions', 'mathlib4-merge-conflict-bot'] nobody
2-62671
2 days ago
unknown
unknown
33877 joelriou
author:joelriou
feat(CategoryTheory/Category/Preorder): isIso_homOfLE We add the lemma `isIso_homOfLE` which shows that `homOfLE` is an isomorphism when `x = y`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory 6/0 Mathlib/CategoryTheory/Category/Preorder.lean 1 9 ['github-actions', 'joelriou', 'vihdzp'] nobody
2-61544
2 days ago
2-55052
2 days ago
2-54872
2 days
33886 joelriou
author:joelriou
feat(CategoryTheory/Triangulated): functors to `Triangle` We introduce constructors for natural transformations and natural isomorphisms between functors to the category of triangles. This will be used in the formalization of spectral sequences #33842. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory 76/0 Mathlib/CategoryTheory/Triangulated/Basic.lean 1 1 ['github-actions'] nobody
2-60032
2 days ago
2-48563
2 days ago
2-48383
2 days
33887 joelriou
author:joelriou
feat(CategoryTheory/Triangulated): fully faithful triangulated functors A fully faithful triangulated functor preserves and reflects distinguished triangles. If the target category satisfies the octahedron axiom (i.e. the category is triangulated), then the source category also is. This is part of the formalization of spectral sequences #33842. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory 45/0 Mathlib/CategoryTheory/Triangulated/Functor.lean 1 1 ['github-actions'] nobody
2-59814
2 days ago
2-47816
2 days ago
2-47636
2 days
33866 robin-carlier
author:robin-carlier
fix(AlgebraicTopology/SimplicialNerve): make `SimplicialThickening` a one field structure When debugging #33822, a build failure occured in `AlgebraicTopology/SimplicialNerve`, which was due to a bad instance: linear orders have an automatic `Category` instance. Thus, recording a `LinearOrder` instance on `SimplicialThickening J` (a type alias for `J` when `J` is a linear order) would conflict with the second `Category` instance put later on that type (where the homs are the type of paths). This is fixed by making `SimplicialThickening J` a one-field structure. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebraic-topology t-category-theory 12/13 Mathlib/AlgebraicTopology/SimplicialNerve.lean 1 1 ['github-actions'] dagurtomas
assignee:dagurtomas
2-58752
2 days ago
2-54004
2 days ago
2-53824
2 days
33888 joelriou
author:joelriou
feat(CategoryTheory/Shift): more API for NatTrans.CommShift We introduce a structure `NatTrans.CommShiftCore` which allows to state that a natural transformation is compatible with shifts in a specific degree. We obtain a few additional results, including that it we have a natural isomorphism `e : F ⋙ G ≅ H` with `G` fully faithful, then the functor `F` commutes with shifts by `A` if `G` and `H` do. This is part of a formalization of spectral sequences #33842. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory 243/1 Mathlib/CategoryTheory/NatIso.lean,Mathlib/CategoryTheory/Shift/CommShift.lean 2 1 ['github-actions'] nobody
2-58429
2 days ago
2-40657
2 days ago
2-40477
2 days
33677 JovanGerb
author:JovanGerb
feat: A linter for instances that overlap on data This PR defines a linter for overlapping instances in declarations. We want to warn users about this, because it leads to local instance diamonds. TODO - expand documentation - Ideally, the linter would be active at all times, included in the standard linter set, and it should also be able to fire on partial declarations, since it only works with the type of the declaration. closes: https://github.com/mathlib-initiative/TaskList/issues/15 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-linter 70/0 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter/OverlappingInstances.lean 3 2 ['euprunin', 'github-actions'] nobody
2-57658
2 days ago
unknown
unknown
33803 erdOne
author:erdOne
feat(RingTheory): integral closure commutes with standard etale basechange --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-ring-theory large-import 260/3 Mathlib/Algebra/Polynomial/Degree/Operations.lean,Mathlib/RingTheory/Etale/Basic.lean,Mathlib/RingTheory/Etale/StandardEtale.lean,Mathlib/RingTheory/Localization/Integral.lean,Mathlib/RingTheory/Smooth/IntegralClosure.lean 5 1 ['github-actions'] nobody
2-54980
2 days ago
2-38586
2 days ago
2-38406
2 days
30985 erdOne
author:erdOne
feat(AlgbraicGeometry), `Hom(-, X)` commutes with inverse limits for schemes of finite presentation --- - [ ] depends on: #30988 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebraic-geometry 208/0 Mathlib/AlgebraicGeometry/AffineScheme.lean,Mathlib/AlgebraicGeometry/AffineTransitionLimit.lean,Mathlib/CategoryTheory/Filtered/Basic.lean,Mathlib/Topology/Sets/OpenCover.lean 4 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
2-54300
2 days ago
2-38868
2 days ago
2-38688
2 days
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra delegated
label:t-algebra$
18/9 Mathlib/Algebra/Group/Units/Hom.lean,Mathlib/AlgebraicGeometry/Scheme.lean,Mathlib/Geometry/RingedSpace/LocallyRingedSpace.lean,Mathlib/Geometry/RingedSpace/OpenImmersion.lean,Mathlib/RingTheory/LocalRing/ResidueField/Basic.lean 5 14 ['adomani', 'alreadydone', 'erdOne', 'eric-wieser', 'github-actions', 'jcommelin', 'leanprover-community-bot-assistant', 'mathlib-bors', 'mathlib4-merge-conflict-bot', 'vihdzp'] mattrobball
assignee:mattrobball
2-53729
2 days ago
58-2152
58 days ago
14-54827
14 days
33532 vihdzp
author:vihdzp
feat(RingTheory/Valuation/ValuativeRel): introduce `=ᵥ` relation Of course, the characterizing property is that for any compatible valuation, `x =ᵥ y` is equivalent to `v x = v y`. --- I haven't yet introduced too much API. I'll be using this on the CGT repo in order to define a `ValuativeRel Surreal` instance compatible with `ArchimedeanClass.mk`. If there's any API I'm missing, I'll upstream it in a subsequent PR. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-ring-theory 70/14 Mathlib/RingTheory/Valuation/ValuativeRel/Basic.lean 1 6 ['erdOne', 'github-actions', 'vihdzp'] erdOne
assignee:erdOne
2-53221
2 days ago
2-53221
2 days ago
9-15977
9 days
33810 dupuisf
author:dupuisf
feat: add instances of `LawfulInv` --- - [ ] depends on: #33441 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP blocked-by-other-PR 187/22 Mathlib/Algebra/GroupWithZero/Defs.lean,Mathlib/Algebra/GroupWithZero/Invertible.lean,Mathlib/Algebra/GroupWithZero/Units/Basic.lean,Mathlib/Analysis/CStarAlgebra/CStarMatrix.lean,Mathlib/LinearAlgebra/Matrix/NonsingularInverse.lean,Mathlib/LinearAlgebra/Matrix/PosDef.lean,Mathlib/RingTheory/DividedPowers/Padic.lean,Mathlib/Topology/Algebra/Module/Equiv.lean,Mathlib/Topology/ContinuousMap/Bounded/Basic.lean 9 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
2-52966
2 days ago
unknown
unknown
32880 0xTerencePrime
author:0xTerencePrime
feat(Analysis/Asymptotics): define subpolynomial growth ## Main definitions * `Asymptotics.IsSubpolynomial l f g`: A function `f` has subpolynomial growth with respect to `g` along filter `l` if `f = O(1 + ‖g‖^k)` for some natural `k`. ## Main results * `IsSubpolynomial.const`: Constant functions have subpolynomial growth * `IsSubpolynomial.id`: Identity has subpolynomial growth * `IsSubpolynomial.add`: Closure under addition * `IsSubpolynomial.neg`: Closure under negation * `IsSubpolynomial.sub`: Closure under subtraction * `IsSubpolynomial.mul`: Closure under multiplication * `IsSubpolynomial.pow`: Closure under powers * `isSubpolynomial_iff_one_add`: Equivalence with `(1 + ‖g‖)^k` formulation * `IsSubpolynomial.uniform`: Uniform bounds for finite families ## Implementation notes The definition uses `1 + ‖g‖^k` rather than `(1 + ‖g‖)^k` as the primary form, with the equivalence established in `isSubpolynomial_iff_one_add`. Four private auxiliary lemmas handle the key inequalities needed for closure proofs. Closes #32658 awaiting-author t-analysis new-contributor 185/0 Mathlib.lean,Mathlib/Analysis/Asymptotics/Subpolynomial.lean 2 28 ['0xTerencePrime', 'ADedecker', 'github-actions', 'j-loreaux'] ADedecker
assignee:ADedecker
2-52365
2 days ago
3-33823
3 days ago
22-12319
22 days
33891 Komyyy
author:Komyyy
refactor: make `Nat.Partrec` protected `Nat.Primrec` is protected to avoid confusion with `Primrec`, but `Nat.Partrec` is not. Furthermore, `Nat.Partrec` is a definition in recursion theory, so frequently used under `open Nat`, and as it is an auxiliary definition of `Partrec`, confusion is particularly problematic. In this PR, we make `Nat.Partrec` protected. --- For reviewers; what I confirmed: * Searched for `Partrec` and confirmed that there are no more places that should be replaced with `Nat.Partrec`. * Searched for `_root_.Partrec` and replaced **as many as possible** with `Partrec`. (The reason not all were replaced is that `Nat.Partrec.lemma_name` and `Partrec.lemma_name` conflict.) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-computability 26/24 Mathlib/Computability/Halting.lean,Mathlib/Computability/Partrec.lean,Mathlib/Computability/PartrecCode.lean 3 1 ['github-actions'] nobody
2-51402
2 days ago
2-37733
2 days ago
2-37553
2 days
33850 YuvalFilmus
author:YuvalFilmus
feat(Chebyshev/ChebyshevGauss): Chebyshev–Gauss formula We prove the Chebyshev–Gauss quadrature formula, which reduces an integral with respect to the Chebyshev weight function to a finite sum. --- - [ ] depends on: #33676 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis blocked-by-other-PR 305/0 Mathlib.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Chebyshev/ChebyshevGauss.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Chebyshev/Orthogonality.lean 3 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
2-47360
2 days ago
unknown
unknown
33843 euprunin
author:euprunin
chore: golf using `grind` and `simp` --- The goal of this golfing PR is to decrease the number of times lemmas are called explicitly (replacing calls to lemmas with calls to tactics). Any decrease in compilation time is a welcome side effect, although it is not a primary objective. Trace profiling results (shown if ≥10 ms before or after): * `ComplexShape.exists_distinct_prev_or`: <10 ms before, 22 ms after * `ComplexShape.exists_distinct_next_or`: <10 ms before, 43 ms after * `DFinsupp.filter_ne_eq_erase'`: <10 ms before, 23 ms after * `List.Pairwise.rel_head_tail`: <10 ms before, 42 ms after * `List.Pairwise.rel_head_of_rel_head_head`: <10 ms before, 63 ms after * `EuclideanGeometry.oangle_eq_oangle_rev_of_two_zsmul_eq_of_angle_eq_pi_div_two`: 78 ms before, <10 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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 7/26 Mathlib/Algebra/Homology/HasNoLoop.lean,Mathlib/Data/DFinsupp/Defs.lean,Mathlib/Data/List/Pairwise.lean,Mathlib/Geometry/Euclidean/Angle/Oriented/RightAngle.lean 4 4 ['Komyyy', 'github-actions'] nobody
2-45040
2 days ago
3-60618
3 days ago
3-60438
3 days
33826 euprunin
author:euprunin
chore: golf using `grind` --- The goal of this golfing PR is to decrease the number of times lemmas are called explicitly (replacing calls to lemmas with calls to tactics). Any decrease in compilation time is a welcome side effect, although it is not a primary objective. Trace profiling results (shown if ≥10 ms before or after): * `List.IsChain.tail`: <10 ms before, 12 ms after * `List.IsChain.cons_of_ne_nil`: 12 ms before, 21 ms after * `List.isChain_attachWith`: 148 ms before, 186 ms after * `List.orderedInsert_erase`: 35 ms before, 73 ms after * `PFunctor.Approx.head_succ'`: 24 ms before, 57 ms after * `not_monotone_not_antitone_iff_exists_le_le`: 40 ms before, 119 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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 7/76 Mathlib/Data/List/Chain.lean,Mathlib/Data/List/Sort.lean,Mathlib/Data/PFunctor/Univariate/M.lean,Mathlib/Order/Monotone/Basic.lean 4 3 ['euprunin', 'github-actions', 'urkud'] nobody
2-45025
2 days ago
4-40202
4 days ago
4-40022
4 days
33897 ADedecker
author:ADedecker
feat(HereditarilyLindelof): review and expand API --- I wrote some of these as suggestions to #31180. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology 54/14 Mathlib/Analysis/Meromorphic/Basic.lean,Mathlib/MeasureTheory/Measure/Support.lean,Mathlib/Topology/Compactness/Lindelof.lean 3 1 ['github-actions'] nobody
2-44274
2 days ago
unknown
unknown
33864 Timeroot
author:Timeroot
feat(Computability/Primrec): Proving several Nat arithmetic functions are primrec Prove that gcd, lcm, coprimality, divisiblity, primality, factorial, descending factorial, powers, and various logarithms are all primitive recursive. Co-authored-by: Aristotle Harmonic <[aristotle-harmonic@harmonic.fun](mailto:aristotle-harmonic@harmonic.fun)> large-import 195/4 Mathlib.lean,Mathlib/Computability/Primrec.lean,Mathlib/Computability/Primrec/List.lean,Mathlib/Computability/Primrec/Nat.lean,Mathlib/Data/Nat/Log.lean 5 5 ['eric-wieser', 'github-actions', 'mathlib4-merge-conflict-bot'] nobody
2-44024
2 days ago
2-26141
2 days ago
2-25961
2 days
33778 ADedecker
author:ADedecker
feat: on a Hereditarily Lindelöf space, any family of lower semicontinuous function admits a countable subfamily with same supremum --- - [ ] depends on: #33897 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology blocked-by-other-PR 168/14 Mathlib.lean,Mathlib/Analysis/Meromorphic/Basic.lean,Mathlib/MeasureTheory/Measure/Support.lean,Mathlib/Topology/Compactness/Lindelof.lean,Mathlib/Topology/Semicontinuity/Lindelof.lean,docs/references.bib 6 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
2-43585
2 days ago
unknown
unknown
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 t-topology 116/0 Mathlib.lean,Mathlib/AlgebraicTopology/FundamentalGroupoid/SemilocallySimplyConnected.lean,Mathlib/Topology/Path.lean 3 11 ['ADedecker', 'alreadydone', 'github-actions', 'jcommelin', 'kim-em', 'mathlib4-merge-conflict-bot'] jcommelin
assignee:jcommelin
2-41876
2 days ago
7-2919
7 days ago
50-52559
50 days
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-category-theory 210/0 Mathlib/Algebra/Homology/DerivedCategory/Ext/Map.lean,Mathlib/Algebra/Homology/DerivedCategory/ShortExact.lean,Mathlib/Algebra/Homology/HomotopyCategory/Pretriangulated.lean,Mathlib/Algebra/Homology/HomotopyCategory/ShortExact.lean 4 11 ['Thmoas-Guan', 'github-actions', 'joelriou', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] eric-wieser
assignee:eric-wieser
2-39351
2 days ago
2-39351
2 days ago
6-48647
6 days
33838 chainstart
author:chainstart
feat(NumberTheory): add unitary divisor sum function ## Summary This PR introduces the unitary divisor sum function σ* to Mathlib and proves that no odd unitary perfect numbers exist. ## Main Definitions - `Nat.UnitaryDivisor d n`: A divisor `d` of `n` is unitary if `gcd(d, n/d) = 1` - `Nat.unitaryDivisors n`: The `Finset` of all unitary divisors of `n` - `Nat.unitaryDivisorSum n` (notation `σ*`): Sum of all unitary divisors - `Nat.UnitaryPerfect n`: `n` is unitary perfect if `σ*(n) = 2n` ## Main Theorems **Multiplicativity:** - `unitaryDivisorSum_mul`: For coprime `m`, `n`, `σ*(mn) = σ*(m) · σ*(n)` - Proved via explicit bijection between unitary divisors of `mn` and pairs of unitary divisors **Prime Powers:** - `unitaryDivisors_prime_pow`: The unitary divisors of `p^k` are exactly `{1, p^k}` - `unitaryDivisorSum_prime_pow`: For prime `p` and `k ≥ 1`, `σ*(p^k) = p^k + 1` **Unitary Perfect Numbers:** - `no_odd_unitary_perfect`: There are no odd unitary perfect numbers > 1 (Subbarao-Warren 1966) - `UnitaryPerfect.even`: Every unitary perfect number is even - `UnitaryPerfect.eq_two_pow_mul_odd`: Every unitary perfect number has form `2^a · k` with `a ≥ 1`, `k` odd ## Mathematical Background A unitary perfect number is a positive integer `n` such that the sum of its unitary divisors equals `2n`. This generalizes the classical perfect numbers. Only five unitary perfect numbers are known: 6, 60, 90, 87360, and one with 24 digits. The main theorem (no odd unitary perfect numbers) was originally proved by Subbarao & Warren (1966) using prime factorization arguments. Our formalization uses `Nat.recOnPrimeCoprime` for structural induction. ## References - Subbarao, M. V., & Warren, L. J. (1966). Unitary perfect numbers. *Canadian Mathematical Bulletin*, 9(2), 147-153. - Wall, C. R. (1975). The fifth unitary perfect number. *Canadian Mathematical Bulletin*, 18(1), 115-122. ## Code Statistics - **Files**: 2 - **Lines**: ~520 - **Theorems**: 21 public declarations - **Sorry count**: 0 ## Checklist - [x] All theorem names follow mathlib conventions - [x] All lines ≤ 100 characters - [x] All public theorems have docstrings - [x] No `sorry` or `admit` - [x] Code builds successfully - [ ] CI tests pass (awaiting verification) new-contributor t-number-theory 557/0 Mathlib.lean,Mathlib/NumberTheory/UnitaryDivisor.lean,Mathlib/NumberTheory/UnitaryPerfect.lean 3 5 ['SnirBroshi', 'chainstart', 'github-actions'] nobody
2-38283
2 days ago
2-54106
2 days ago
3-72342
3 days
33477 mcdoll
author:mcdoll
refactor(Algebra): add type-classes for algebraic properties of `FunLike` --- Zulip discussion: [#mathlib4 > Refactoring algebraic properties of bundled maps](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Refactoring.20algebraic.20properties.20of.20bundled.20maps/with/566142461) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict large-import 721/208 Mathlib.lean,Mathlib/Algebra/BigOperators/Pi.lean,Mathlib/Algebra/Category/Grp/Colimits.lean,Mathlib/Algebra/Category/Grp/EpiMono.lean,Mathlib/Algebra/Category/ModuleCat/Topology/Basic.lean,Mathlib/Algebra/DirectSum/Ring.lean,Mathlib/Algebra/FiveLemma.lean,Mathlib/Algebra/Group/Hom/Basic.lean,Mathlib/Algebra/Group/Hom/Defs.lean,Mathlib/Algebra/Group/Hom/End.lean,Mathlib/Algebra/Group/Hom/FunLike.lean,Mathlib/Algebra/Group/Hom/Instances.lean,Mathlib/Algebra/Group/Pi/Lemmas.lean,Mathlib/Algebra/GroupWithZero/Hom.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/ExactSequences.lean,Mathlib/Algebra/Homology/HomotopyCategory/HomComplexCohomology.lean,Mathlib/Algebra/Homology/ShortComplex/Ab.lean,Mathlib/Algebra/Module/CharacterModule.lean,Mathlib/Algebra/Module/End.lean,Mathlib/Algebra/Module/FunLike.lean,Mathlib/Algebra/Module/GradedModule.lean,Mathlib/Algebra/Module/Hom.lean,Mathlib/Algebra/Polynomial/HasseDeriv.lean,Mathlib/Analysis/Distribution/FourierSchwartz.lean,Mathlib/Analysis/Distribution/SchwartzSpace.lean,Mathlib/Analysis/Fourier/LpSpace.lean,Mathlib/Analysis/LocallyConvex/PointwiseConvergence.lean,Mathlib/Analysis/Normed/Group/Hom.lean,Mathlib/Analysis/Normed/Group/SemiNormedGrp/Kernels.lean,Mathlib/Analysis/Normed/Lp/ProdLp.lean,Mathlib/Analysis/Normed/Module/FiniteDimension.lean,Mathlib/Analysis/Normed/Operator/ContinuousAlgEquiv.lean,Mathlib/Analysis/RCLike/Basic.lean,Mathlib/CategoryTheory/Action/Basic.lean,Mathlib/GroupTheory/GroupExtension/Defs.lean,Mathlib/LinearAlgebra/Determinant.lean,Mathlib/LinearAlgebra/TensorProduct/Basic.lean,Mathlib/NumberTheory/MulChar/Basic.lean,Mathlib/RepresentationTheory/Basic.lean,Mathlib/RingTheory/IntegralDomain.lean,Mathlib/RingTheory/RootsOfUnity/Basic.lean,Mathlib/Topology/Algebra/Group/Basic.lean,Mathlib/Topology/Algebra/Module/StrongTopology.lean 43 7 ['github-actions', 'leanprover-radar', 'mathlib4-merge-conflict-bot', 'mcdoll', 'plp127'] nobody
2-37758
2 days ago
unknown
unknown
33905 plp127
author:plp127
chore(Order/RelClasses): name arguments of recursors Name the motive `motive` and name the minor premises something descriptive. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order 12/9 Mathlib/Order/RelClasses.lean 1 1 ['github-actions'] nobody
2-34619
2 days ago
unknown
unknown
33613 DavidLedvinka
author:DavidLedvinka
feat(Probability): `UniformOn_univ_instIsProbabilityMeasure` It is convenient to have an instance of `IsProbabilityMeasure` on a uniform distribution on `.univ` (to avoid the need for `haveI` statements). There is perhaps an argument for `abbrev uniform := uniformOn (.univ : Set Ω)` but I have not implemented this in this PR. t-measure-probability 11/0 Mathlib/Probability/UniformOn.lean 1 5 ['DavidLedvinka', 'Ruben-VandeVelde', 'github-actions'] kex-y
assignee:kex-y
2-31266
2 days ago
5-71342
5 days ago
7-69282
7 days
33736 fbarroero
author:fbarroero
feat(RingTheory/Polynomial/GaussNorm): The `gaussNorm` is an absolute value if `v` is a nonarchimedean absolute value We prove ``` Polynomial.gaussNorm_isAbsoluteValue {c : ℝ} {R : Type*} [Ring R] {v : AbsoluteValue R ℝ} (hna : IsNonarchimedean v) (hc : 0 < c) : IsAbsoluteValue (gaussNorm v c) ``` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 194/7 Mathlib/Algebra/Order/AbsoluteValue/Basic.lean,Mathlib/Algebra/Order/Ring/IsNonarchimedean.lean,Mathlib/RingTheory/Polynomial/GaussNorm.lean 3 4 ['copilot-pull-request-reviewer', 'github-actions'] ADedecker
assignee:ADedecker
2-31264
2 days ago
5-60767
5 days ago
5-60587
5 days
33743 jcommelin
author:jcommelin
ci: add automated commit verification This PR adds verification for "x: " commits that checks whether re-running the command produces the same tree. Written with the help of Claude Code. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) CI 406/28 .github/workflows/commit_verification.yml,scripts/README.md,scripts/verify_commits.sh,scripts/verify_commits_summary.sh 4 6 ['Vierkantor', 'github-actions', 'jcommelin'] joneugster
assignee:joneugster
2-31263
2 days ago
7-3255
7 days ago
7-3075
7 days
33782 tb65536
author:tb65536
refactor(RingTheory/Lasker): create structure for primary decomposition This PR extracts the conclusion of the Lasker-Noether theorem into a separate predicate, so that (in a follow-up PR), the various properties of the primary decomposition don't have to rewrite the entire three-line predicate each time. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-ring-theory t-algebra
label:t-algebra$
19/6 Mathlib/RingTheory/Lasker.lean 1 7 ['erdOne', 'github-actions', 'tb65536'] chrisflav
assignee:chrisflav
2-31260
2 days ago
4-39747
4 days ago
5-24466
5 days
33784 tb65536
author:tb65536
refactor(Topology/Irreducible): weaken assumptions of `preimage_mem_irreducibleComponents_of_isPreirreducible_fiber` This PR weakens the surjectivity assumption of `preimage_mem_irreducibleComponents_of_isPreirreducible_fiber` to `(t ∩ Set.range f).Nonempty`. I also took the liberty of systematizing the file slightly, so that now there are 6 lemmas: preimage of (preirreducible / irreducible / irreducible component) assuming (preirreducible fibers / open embedding). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology 36/26 Mathlib/Topology/Irreducible.lean 1 1 ['github-actions'] alreadydone
assignee:alreadydone
2-31259
2 days ago
6-27754
6 days ago
6-27574
6 days
33786 hdmkindom
author:hdmkindom
feat(Analysis/Matrix): add Jacobian matrix for matrix-valued functions This PR introduces the Jacobian matrix for matrix-valued functions `F : Matrix m n ℝ → Matrix p q ℝ`. The Jacobian matrix `jacobianMatrix F X` at point `X` is indexed by `(p × q) × (m × n)`, where each entry represents the partial derivative with respect to a basis element. To handle instance-mismatch issues with matrix norms, we use local Frobenius norm instances. mkdir Analysis/Matrix/Jacobian.lean ## Main definitions - `jacobianMatrix F X`: The Jacobian matrix at point `X`, defined by `jacobianMatrix F X (i, k) (j, l) = (fderiv ℝ F X (Matrix.single j l 1)) i k` ## Main theorems - `fderiv_eq_jacobian_mul`: Express the Fréchet derivative as a contraction with the Jacobian - `jacobianMatrix_comp`: Chain rule for Jacobian matrices - `jacobianMatrix_linear`, `jacobianMatrix_id`, `jacobianMatrix_const`: Basic properties - `jacobianMatrix_add`, `jacobianMatrix_smul`: Linearity properties t-analysis new-contributor 219/0 Mathlib.lean,Mathlib/Analysis/Matrix/Jacobian.lean 2 1 ['github-actions'] ADedecker
assignee:ADedecker
2-31257
2 days ago
5-65932
5 days ago
6-10090
6 days
33795 alreadydone
author:alreadydone
feat(Topology/Sheaves): LocalPredicate prerequisite for étalé spaces --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology 417/145 Mathlib/AlgebraicGeometry/Modules/Tilde.lean,Mathlib/AlgebraicGeometry/ProjectiveSpectrum/StructureSheaf.lean,Mathlib/Geometry/Manifold/Sheaf/Smooth.lean,Mathlib/Logic/Equiv/Basic.lean,Mathlib/Topology/Sheaves/LocalPredicate.lean,Mathlib/Topology/Sheaves/Sheafify.lean,Mathlib/Topology/Sheaves/Stalks.lean 7 1 ['github-actions'] dagurtomas
assignee:dagurtomas
2-31255
2 days ago
5-53320
5 days ago
5-53140
5 days
33862 dupuisf
author:dupuisf
chore(AkraBazzi): golf the main proof This PR significantly shortens the main proof of the Akra-Bazzi theorem, removing an `adaptation_note` in the process. --- - [ ] depends on: #33907 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-analysis blocked-by-other-PR 244/302 Mathlib/Analysis/Asymptotics/Lemmas.lean,Mathlib/Computability/AkraBazzi/AkraBazzi.lean 2 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
2-23067
2 days ago
unknown
unknown
33504 ldct
author:ldct
feat: Add lemmas for DihedralGroup.fintypeHelper Using `fin_cases` to reason about `DihedralGroup` elements exposes the internal `fintypeHelper` instances, which has no exported API ``` example (g : DihedralGroup 3) : (g^6 = 1) := by fin_cases g <;> dsimp -- 6 goals case «0» ⊢ DihedralGroup.fintypeHelper✝ (Sum.inl 0) ^ 6 = 1 ... ``` this PR adds simp lemma that convert them to constructors, which do have API ``` 6 goals case «0» ⊢ 1 ^ 6 = 1 case «1» ⊢ DihedralGroup.r 1 ^ 6 = 1 case «2» ⊢ DihedralGroup.r 2 ^ 6 = 1 ``` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-group-theory 8/0 Mathlib/GroupTheory/SpecificGroups/Dihedral.lean 1 1 ['github-actions', 'tb65536'] nobody
2-12814
2 days ago
12-16151
12 days ago
12-15971
12 days
33718 erdOne
author:erdOne
feat(RingTheory): predicate for `QuasiFiniteAt` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-ring-theory 267/26 Mathlib/RingTheory/Etale/QuasiFinite.lean,Mathlib/RingTheory/LocalRing/ResidueField/Ideal.lean,Mathlib/RingTheory/Localization/AtPrime/Basic.lean,Mathlib/RingTheory/QuasiFinite/Basic.lean 4 9 ['chrisflav', 'erdOne', 'github-actions'] nobody
2-6153
2 days ago
2-6153
2 days ago
4-22313
4 days
33757 fpvandoorn
author:fpvandoorn
feat: remove decidability instances on sets or ideals * We have the rule that you should assume decidability instead of opening the classical locale. However, in places where there cannot ever be a reasonable decidable instance, I think we can relax this rule. * This PR updates the corresponding library note, and removes `DecidableEq` instances on `Set` and `Ideal` * This looks a lot cleaner IMO, and the decidability assumptions are silly: assuming that `Set α` has decidable for an inhabited type `α` is equivalent to assuming that all propositions are decidable. Similarly for `Ideal R` for a nontrivial ring `R`. * This has one downside: if a lemma uses classical logic to infer decidability for its statement, then all lemmas that use this lemma also have to do this, otherwise they will deal with decidability type mismatches --- This was motivated by seeing some code from @mariainesdff's repos with such decidability arguments. @mariainesdff, do you think this PR would make your code a bit nicer? [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 57/32 Mathlib/Algebra/Module/DedekindDomain.lean,Mathlib/Algebra/Module/PID.lean,Mathlib/Logic/Basic.lean,Mathlib/MeasureTheory/SetSemiring.lean,Mathlib/NumberTheory/RamificationInertia/Basic.lean,Mathlib/Order/PartialSups.lean,Mathlib/RingTheory/DedekindDomain/Factorization.lean,Mathlib/RingTheory/DedekindDomain/Ideal/Lemmas.lean,Mathlib/RingTheory/Ideal/Basic.lean,Mathlib/RingTheory/Invariant/Basic.lean,Mathlib/RingTheory/Lasker.lean,Mathlib/RingTheory/Valuation/ValuationRing.lean 12 5 ['github-actions', 'plp127', 'vihdzp'] nobody
2-5221
2 days ago
6-61042
6 days ago
6-60862
6 days
33780 ooovi
author:ooovi
feat(Geometry/Convex/Cone): lineality space of pointed cones Define the lineality space `PointedCone.lineal` as the submodule `C ⊓ -C`. Prove that it is the largest submodule of the cone, which is sometimes used as an alternative definition. Co-authored-by: Martin Winter --- dependency of #33664 - [x] depends on #33761 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-convex-geometry 41/1 Mathlib/Geometry/Convex/Cone/Pointed.lean 1 6 ['eric-wieser', 'github-actions', 'martinwintermath', 'mathlib4-merge-conflict-bot'] nobody
2-4344
2 days ago
unknown
unknown
33664 ooovi
author:ooovi
feat(Geometry/Convex/Cone/Pointed): face lattice of pointed cones - Create a subdirectory in `Cone` for pointed cones and move existing files there. - Define `PointedCone.IsFaceOf`, for a pointed cone being a face of another pointed cone. - Prove some basic properties, that faces are extreme sets of their cone, and how they behave under intersection, map and product operations. - Define `Face` by bundling the `IsFaceOf` structure, and show the complete lattice structure on it. - Prove that taking the product of two faces is an order isomorphism. Co-authored-by: Martin Winter --- - [ ] depends on #33780 for the definition of the lineal space [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) file-removed awaiting-author t-convex-geometry 542/10 Mathlib.lean,Mathlib/Analysis/Convex/Cone/Basic.lean,Mathlib/Analysis/Convex/Cone/Closure.lean,Mathlib/Analysis/Convex/Cone/Dual.lean,Mathlib/Geometry/Convex/Cone/Pointed/Basic.lean,Mathlib/Geometry/Convex/Cone/Pointed/Dual.lean,Mathlib/Geometry/Convex/Cone/Pointed/Face/Basic.lean,Mathlib/Geometry/Convex/Cone/Pointed/Face/Lattice.lean,Mathlib/Geometry/Convex/Cone/Pointed/TensorProduct.lean 9 85 ['YaelDillies', 'eric-wieser', 'github-actions', 'martinwintermath', 'mathlib4-merge-conflict-bot', 'ooovi'] nobody
2-2911
2 days ago
8-72727
8 days ago
0-4399
1 hour
33878 xroblot
author:xroblot
feat(MulChar): generalize duality results on finite abelian groups to multiplicative characters --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-number-theory 324/21 Mathlib/Algebra/Group/Subgroup/Map.lean,Mathlib/Algebra/Group/Submonoid/BigOperators.lean,Mathlib/Algebra/Group/Submonoid/Operations.lean,Mathlib/Algebra/Group/Submonoid/Units.lean,Mathlib/GroupTheory/Exponent.lean,Mathlib/GroupTheory/FiniteAbelian/Duality.lean,Mathlib/GroupTheory/QuotientGroup/Basic.lean,Mathlib/NumberTheory/MulChar/Basic.lean,Mathlib/NumberTheory/MulChar/Duality.lean,Mathlib/NumberTheory/MulChar/Lemmas.lean,Mathlib/RingTheory/RootsOfUnity/Basic.lean 11 1 ['github-actions'] nobody
2-2355
2 days ago
1-84447
1 day ago
1-84267
1 day
33893 MichaelStollBayreuth
author:MichaelStollBayreuth
feat(NumberTheory/Height): heights of tuples and finsupps This is the second PR on heights. We add the definition of the height of a tuple of field elements (and of finitely supported maps into the field) and prove some properties, for example the invariance under scaling by a nonzero field element. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-number-theory 210/0 Mathlib/NumberTheory/Height/Basic.lean,Mathlib/NumberTheory/Height/Instances.lean 2 1 ['github-actions'] nobody
2-249
2 days ago
2-249
2 days ago
2-69
2 days
33355 0xTerencePrime
author:0xTerencePrime
feat(Combinatorics/SimpleGraph/Connectivity): define vertex connectivity This PR introduces the foundations of vertex connectivity for simple graphs, providing a counterpart to the edge connectivity theory in #32870. ### Main definitions - `SimpleGraph.IsVertexReachable`: vertices remain reachable after removing strictly fewer than `k` other vertices. - `SimpleGraph.IsVertexConnected`: a graph is `k`-vertex-connected if its order is strictly greater than `k` and any two distinct vertices are `k`-vertex-reachable. Includes basic characterizations for $k=0$ and $k=1$, along with monotonicity lemmas (`anti` and `mono`). new-contributor t-combinatorics 154/0 Mathlib.lean,Mathlib/Combinatorics/SimpleGraph/Connectivity/VertexConnectivity.lean,Mathlib/Combinatorics/SimpleGraph/IsolateVerts.lean 3 105 ['0xTerencePrime', 'SnirBroshi', 'YaelDillies', 'github-actions', 'vihdzp'] nobody
1-84586
1 day ago
2-52899
2 days ago
16-77184
16 days
33802 stepan2698-cpu
author:stepan2698-cpu
feat: Schur's lemma for monoid representations Adds an algebra instance on the set of intertwining maps. Proves various versions of Schur's lemma for monoid representations and proves that a finite-dimensional irreducible representation of a commutative monoid is one-dimensional. --- - [ ] depends on: #32856 - [ ] depends on: #33221 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra blocked-by-other-PR
label:t-algebra$
458/11 Mathlib.lean,Mathlib/RepresentationTheory/Intertwining.lean,Mathlib/RepresentationTheory/Irreducible.lean,Mathlib/RepresentationTheory/Subrepresentation.lean 4 3 ['alreadydone', 'github-actions', 'mathlib4-dependent-issues-bot'] ocfnash
assignee:ocfnash
1-78840
1 day ago
1-80476
1 day ago
3-56780
3 days
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). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict file-removed awaiting-author t-algebra
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 11 ['Ruben-VandeVelde', 'YaelDillies', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-merge-conflict-bot', 'riccardobrasca'] riccardobrasca
assignee:riccardobrasca
1-76839
1 day ago
105-83937
105 days ago
13-72205
13 days
29186 winstonyin
author:winstonyin
feat: IsIntegralCurve for solutions to ODEs I define `IsIntegralCurve` etc. for solutions to ODEs on vector spaces. The translation and scaling lemmas are also included. This parallels `IsMIntegralCurve` etc. for manifolds. Moved from #26534. - [x] depends on: #26563 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-dynamics t-differential-geometry t-analysis awaiting-author 305/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 20 ['github-actions', 'grunweg', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'mcdoll', 'sgouezel', 'winstonyin'] sgouezel
assignee:sgouezel
1-76483
1 day ago
1-76483
1 day ago
62-62827
62 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) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
398/185 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/Translate/ToAdditive.lean 30 13 ['JovanGerb', 'adomani', 'alreadydone', 'bryangingechen', 'github-actions', 'mathlib4-merge-conflict-bot'] bryangingechen
assignee:bryangingechen
1-76298
1 day ago
1-72585
1 day ago
99-49660
99 days
33842 joelriou
author:joelriou
feat(Algebra/Homology): spectral sequences This PR introduces spectral sequences. It contains two mostly independent developments: 1. The construction of the spectral object attached to objects in a triangulated category `C` equipped with a t-structure; 2. The definition of a category of spectral sequences and the construction of the spectral sequence attached to a spectral objects indexed by the extended integers (the integers with +/- infinity) in an abelian category. After these additions, we have two ways to construct a spectral object in triangulated categories (the spectral object attached to a filtered complex, and the spectral object attached to a t-structure 1.). After applying a homological functor to these spectral objects, we obtain a spectral object in an abelian category, and the construction 2. allows to define spectral sequences. In this PR, we do not study the stabilization and convergence of spectral sequences, which require more developments. The computation of the first page of the constructed spectral sequences would be an easy addition. The mathematical material is discussed in https://hal.science/hal-04546712v5 (§5.4.1 and §5.4.4). --- 3. Prerequisites: - [ ] depends on: #33874 - [ ] depends on: #33875 - [ ] depends on: #33876 - [ ] depends on: #33877 - [ ] depends on: #33879 - [ ] depends on: #33880 - [ ] depends on: #33881 - [ ] depends on: #33437 - [ ] depends on: #33883 - [ ] depends on: #33886 - [ ] depends on: #33887 - [ ] depends on: #33888 - [ ] depends on: #33890 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR WIP t-category-theory large-import 7236/60 Mathlib.lean,Mathlib/Algebra/Homology/ExactSequence.lean,Mathlib/Algebra/Homology/ExactSequenceFour.lean,Mathlib/Algebra/Homology/ShortComplex/Abelian.lean,Mathlib/Algebra/Homology/ShortComplex/Basic.lean,Mathlib/Algebra/Homology/ShortComplex/Exact.lean,Mathlib/Algebra/Homology/ShortComplex/Homology.lean,Mathlib/Algebra/Homology/ShortComplex/LeftHomology.lean,Mathlib/Algebra/Homology/ShortComplex/RightHomology.lean,Mathlib/Algebra/Homology/SpectralObject/Basic.lean,Mathlib/Algebra/Homology/SpectralObject/Cycles.lean,Mathlib/Algebra/Homology/SpectralObject/Differentials.lean,Mathlib/Algebra/Homology/SpectralObject/HasSpectralSequence.lean,Mathlib/Algebra/Homology/SpectralObject/Homology.lean,Mathlib/Algebra/Homology/SpectralObject/Page.lean,Mathlib/Algebra/Homology/SpectralObject/SpectralSequence.lean,Mathlib/Algebra/Homology/SpectralSequence/Basic.lean,Mathlib/Algebra/Homology/SpectralSequence/ComplexShape.lean,Mathlib/CategoryTheory/Category/Preorder.lean,Mathlib/CategoryTheory/ComposableArrows/Basic.lean,Mathlib/CategoryTheory/ComposableArrows/Four.lean,Mathlib/CategoryTheory/ComposableArrows/Three.lean,Mathlib/CategoryTheory/ComposableArrows/Two.lean,Mathlib/CategoryTheory/Limits/Shapes/Equalizers.lean,Mathlib/CategoryTheory/Limits/Shapes/Products.lean,Mathlib/CategoryTheory/Limits/Shapes/ZeroObjects.lean,Mathlib/CategoryTheory/NatIso.lean,Mathlib/CategoryTheory/ObjectProperty/ContainsZero.lean,Mathlib/CategoryTheory/ObjectProperty/FullSubcategory.lean,Mathlib/CategoryTheory/ObjectProperty/Shift.lean,Mathlib/CategoryTheory/Preadditive/AdditiveFunctor.lean,Mathlib/CategoryTheory/Shift/CommShift.lean,Mathlib/CategoryTheory/Triangulated/Basic.lean,Mathlib/CategoryTheory/Triangulated/Functor.lean,Mathlib/CategoryTheory/Triangulated/Pretriangulated.lean,Mathlib/CategoryTheory/Triangulated/Subcategory.lean,Mathlib/CategoryTheory/Triangulated/TStructure/Basic.lean,Mathlib/CategoryTheory/Triangulated/TStructure/ETrunc.lean,Mathlib/CategoryTheory/Triangulated/TStructure/Induced.lean,Mathlib/CategoryTheory/Triangulated/TStructure/SpectralObject.lean,Mathlib/CategoryTheory/Triangulated/TStructure/TruncLEGT.lean,Mathlib/CategoryTheory/Triangulated/TStructure/TruncLTGE.lean,Mathlib/Data/EInt/Basic.lean,Mathlib/Order/WithBotTop.lean 44 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
1-72323
1 day ago
unknown
unknown
33675 euprunin
author:euprunin
feat(RingTheory/RingHom): remove unnecessary assumptions in `locally_StableUnderCompositionWithLocalizationAwayTarget` (WIP) --- Marked as WIP pending reviewer confirmation that the assumptions are unnecessary not only logically, but also semantically. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-ring-theory 1/3 Mathlib/RingTheory/RingHom/Locally.lean 1 2 ['euprunin', 'github-actions'] nobody
1-70815
1 day ago
unknown
unknown
33901 martinwintermath
author:martinwintermath
feat(LinearAlgebra/Span): add inter/union/sInf/sSup lemmas for Submodule.span * Add `inter`, `sInf` and `biInter` lemmas for `Submodule.span` * Add `union`, `sSup` and `biUnion` lemmas for `Submodule.span` * Add `@[simp]` to `span_union` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra
label:t-algebra$
25/0 Mathlib/LinearAlgebra/Span/Defs.lean 1 3 ['github-actions', 'themathqueen'] nobody
1-69917
1 day ago
1-63402
1 day ago
1-63222
1 day
32757 AntoineChambert-Loir
author:AntoineChambert-Loir
feat(LinearAlgebra/Transvection): the determinant of a transvection is equal to 1. Prove 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$$. --- - [x] depends on: #31138 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 255/0 Mathlib/LinearAlgebra/Determinant.lean,Mathlib/LinearAlgebra/Transvection.lean 2 10 ['AntoineChambert-Loir', 'alreadydone', 'eric-wieser', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
1-69817
1 day ago
1-64763
1 day ago
23-10004
23 days
33911 YaelDillies
author:YaelDillies
feat(Data/Set/Finite): make simp more powerful From ProofBench --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data 13/9 Archive/Examples/Kuratowski.lean,Mathlib/Data/Finite/Defs.lean,Mathlib/Data/Set/Finite/Basic.lean 3 1 ['github-actions'] nobody
1-69029
1 day ago
1-63190
1 day ago
1-63010
1 day
33903 erdOne
author:erdOne
feat(RingTheory): local structure of monogenic unramified algebras --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-ring-theory large-import 295/3 Mathlib.lean,Mathlib/RingTheory/LocalRing/ResidueField/Polynomial.lean,Mathlib/RingTheory/TensorProduct/Basic.lean,Mathlib/RingTheory/Unramified/Field.lean,Mathlib/RingTheory/Unramified/LocalStructure.lean,Mathlib/RingTheory/Unramified/Locus.lean 6 1 ['github-actions'] nobody
1-68999
1 day ago
1-62711
1 day ago
1-62531
1 day
33318 harahu
author:harahu
doc(Analysis): fix file refs --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis 14/8 Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Note.lean,Mathlib/Analysis/Calculus/FDeriv/Basic.lean,Mathlib/Analysis/Calculus/FDeriv/Defs.lean 3 1 ['euprunin', 'github-actions'] nobody
1-68156
1 day ago
unknown
unknown
33323 harahu
author:harahu
doc(Algebra): fix file refs Address some stale file refs in `Algebra`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
4/3 Mathlib/Algebra/Group/Pointwise/Finset/Interval.lean,Mathlib/Algebra/Module/Submodule/Lattice.lean,Mathlib/Algebra/Order/Module/OrderedSMul.lean 3 5 ['euprunin', 'github-actions', 'harahu', 'mathlib4-merge-conflict-bot'] nobody
1-68122
1 day ago
2-16798
2 days ago
5-34940
5 days
33797 SnirBroshi
author:SnirBroshi
chore(Order/Defs/Unbundled): deprecate `IsTotal` in favor of core's `Std.Total` --- [Mathlib's `IsTotal`](https://leanprover-community.github.io/mathlib4_docs/Mathlib/Order/Defs/Unbundled.html#IsTotal) [Core's `Std.Total`](https://leanprover-community.github.io/mathlib4_docs/Init/Core.html#Std.Total) [Zulip](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Relation.20properties.20duplication/near/544638270) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order 121/107 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/DFinsupp/Lex.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/Real/Basic.lean,Mathlib/Data/Sigma/Lex.lean,Mathlib/Data/Sum/Order.lean,Mathlib/Logic/Encodable/Basic.lean,Mathlib/Order/Antisymmetrization.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/Quotient.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,Mathlib/Topology/Semicontinuity/Basic.lean 33 10 ['SnirBroshi', 'github-actions', 'vihdzp'] nobody
1-67910
1 day ago
1-67979
1 day ago
2-82465
2 days
33028 bjornsolheim
author:bjornsolheim
feat(Geometry/Convex/Cone): minimal and maximal cone tensor products are commutative Prove that the minimal and maximal cone tensor products are commutative. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-convex-geometry 62/0 Mathlib/Geometry/Convex/Cone/TensorProduct.lean,Mathlib/LinearAlgebra/Dual/Lemmas.lean 2 13 ['artie2000', 'bjornsolheim', 'github-actions'] nobody
1-67703
1 day ago
1-60419
1 day ago
27-23982
27 days
27053 tb65536
author:tb65536
feat: Galois group of `x^n - x - 1` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-algebra large-import
label:t-algebra$
405/151 Archive/Wiedijk100Theorems/AbelRuffini.lean,Mathlib/RingTheory/Polynomial/Selmer.lean 2 7 ['AntoineChambert-Loir', 'github-actions', 'mathlib4-merge-conflict-bot'] nobody
1-66980
1 day ago
unknown
unknown
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 - [x] depends on: #30356 - [ ] depends on: #28796 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR t-meta t-differential-geometry 286/87 Mathlib/Analysis/Calculus/ContDiff/Basic.lean,Mathlib/Geometry/Manifold/ContMDiff/Atlas.lean,Mathlib/Geometry/Manifold/Immersion.lean,Mathlib/Geometry/Manifold/IsManifold/ExtChartAt.lean,Mathlib/Geometry/Manifold/LocalSourceTargetProperty.lean,Mathlib/Geometry/Manifold/SmoothEmbedding.lean 6 4 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
1-65799
1 day ago
unknown
unknown
33853 farmanb
author:farmanb
feat(RingTheory/IdealFilter): topologies associated to ideal filters This PR introduces topological structures on a ring arising from an IdealFilter. Main additions: * `IdealFilter.addGroupFilterBasis` and the induced additive group topology. * Under `F.IsUniform`, `IdealFilter.ringFilterBasis` and the induced ring topology. * A characterization of uniform ideal filters in terms of the existence of a `RingFilterBasis` (`isUniform_iff_exists_ringFilterBasis`). * Neighborhood characterizations for both the additive and ring topologies. * A proof that the resulting ring topology is linear (`IsLinearTopology`). The construction follows the standard picture of uniform (Gabriel) filters generating linear topologies on rings, using colon ideals to witness stability under right multiplication. This provides the topological counterpart to the algebraic theory of ideal filters developed in RingTheory/IdealFilter/Basic. --- - [ ] depends on: #33021 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-ring-theory new-contributor blocked-by-other-PR 601/56 Mathlib.lean,Mathlib/RingTheory/Ideal/Colon.lean,Mathlib/RingTheory/Ideal/Oka.lean,Mathlib/RingTheory/IdealFilter/Basic.lean,Mathlib/RingTheory/IdealFilter/Topology.lean,Mathlib/RingTheory/Lasker.lean,Mathlib/RingTheory/Noetherian/OfPrime.lean,Mathlib/RingTheory/PrincipalIdealDomainOfPrime.lean,Mathlib/RingTheory/Support.lean,docs/references.bib 10 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
1-64384
1 day ago
unknown
unknown
33885 WenrongZou
author:WenrongZou
feat(RingTheory/MvPowerSeries): some theorems about expand --- I add some theorems for `MvPowerSeries.expand` to make it reusable. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-ring-theory 87/7 Mathlib/RingTheory/MvPowerSeries/Expand.lean,Mathlib/RingTheory/MvPowerSeries/Substitution.lean,Mathlib/RingTheory/PowerSeries/Expand.lean,Mathlib/RingTheory/PowerSeries/Substitution.lean 4 1 ['github-actions'] nobody
1-62980
1 day ago
1-55409
1 day ago
1-55229
1 day
33793 LTolDe
author:LTolDe
feat(MeasureTheory/Constructions/Polish/Basic): add lemma AnalyticSet.inter_nonempty_of_nowhereMeagre add lemma AnalyticSet.inter_nonempty_of_nowhereMeagre, the main ingredient for the proof of the **Effros' Theorem**, see [#mathlib4 > Effros Theorem](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Effros.20Theorem/with/566543328) introduce definition of a nowhere meagre set --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-measure-probability new-contributor 37/0 Mathlib/MeasureTheory/Constructions/Polish/Basic.lean,Mathlib/Order/Filter/Basic.lean,Mathlib/Topology/GDelta/Basic.lean 3 2 ['MichaelStollBayreuth', 'github-actions'] nobody
1-62655
1 day ago
5-67380
5 days ago
5-67200
5 days
33890 joelriou
author:joelriou
feat(CategoryTheory/Triangulated): distinguished_iff_of_isZero When one of the objects of a triangle is zero, the triangle is distinguished iff the morphism between the other objects is an isomorphism. This will be used in the formalization of spectral sequences #33842. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory 50/1 Mathlib/CategoryTheory/Triangulated/Pretriangulated.lean 1 1 ['github-actions'] nobody
1-60535
1 day ago
1-54310
1 day ago
1-54130
1 day
33908 erdOne
author:erdOne
perf: set `IsScalarTower.right` to high priority --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
2/1 Mathlib/Algebra/Algebra/Defs.lean 1 6 ['erdOne', 'github-actions', 'grunweg', 'leanprover-radar'] nobody
1-60430
1 day ago
1-61313
1 day ago
1-82425
1 day
33746 ster99
author:ster99
feat(Algebra/Module/ZLattice): add lemma `floor b (m + x) = m + floor b x` and similar Prove lemmas corresponding to [Int.floor_intCast_add](https://leanprover-community.github.io/mathlib4_docs/Mathlib/Algebra/Order/Floor/Ring.html#Int.floor_intCast_add) and similar for `ZLattice` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra new-contributor
label:t-algebra$
28/0 Mathlib/Algebra/Module/ZLattice/Basic.lean 1 2 ['github-actions'] nobody
1-60152
1 day ago
1-53523
1 day ago
6-78982
6 days
33917 tb65536
author:tb65536
feat(Algebra/Module/LocalizedModule/Submodule): add `inf` and `sup` API This PR adds some more API for `localized₀` and `localized'`. In particular, we show that localization of submodule distributes over finite intersections and arbitrary unions. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-ring-theory t-algebra
label:t-algebra$
58/1 Mathlib/Algebra/Module/LocalizedModule/Submodule.lean 1 1 ['github-actions'] nobody
1-59262
1 day ago
1-59262
1 day ago
1-59082
1 day
33924 martinwintermath
author:martinwintermath
feat(Order/ModularLattice): add some dual codisjoint lemma for modular lattices Add four codisjoint lemmas dual to existing disjoint lemmas for modular lattices: * Add `codisjoint_inf_right_of_codisjoint_inf_left` * Add `codisjoint_inf_left_of_codisjoint_inf_right` * Add `isCompl_inf_right_of_isCompl_inf_left` * Add `isCompl_inf_left_of_isCompl_inf_right` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order new-contributor 34/13 Mathlib/Order/ModularLattice.lean 1 1 ['github-actions'] nobody
1-58111
1 day ago
1-45151
1 day ago
1-44971
1 day
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 --- - [x] depends on: #30413 - [x] depends on: #30879 - [ ] depends on: #33923 (a 5 line fix) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-differential-geometry t-meta blocked-by-other-PR 577/33 Mathlib/Geometry/Manifold/Instances/UnitsOfNormedAlgebra.lean,Mathlib/Geometry/Manifold/Notation.lean,MathlibTest/DifferentialGeometry/Notation.lean,MathlibTest/DifferentialGeometry/NotationAdvanced.lean,MathlibTest/DifferentialGeometry/NotationSphere.lean 5 12 ['github-actions', 'grunweg', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'thorimur'] thorimur
assignee:thorimur
1-57579
1 day ago
unknown
unknown
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 - [x] depends on: #28853 (for simplicity) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-differential-geometry maintainer-merge 192/21 Mathlib/Analysis/Calculus/ContDiff/Basic.lean,Mathlib/Geometry/Manifold/ContMDiff/Atlas.lean,Mathlib/Geometry/Manifold/Immersion.lean,Mathlib/Geometry/Manifold/IsManifold/ExtChartAt.lean,Mathlib/Geometry/Manifold/LocalSourceTargetProperty.lean,Mathlib/Geometry/Manifold/SmoothEmbedding.lean 6 45 ['chrisflav', 'github-actions', 'grunweg', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] PatrickMassot
assignee:PatrickMassot
1-57567
1 day ago
2-78953
2 days ago
24-68813
24 days
33844 michelsol
author:michelsol
feat: lemmas to change variables in iSup / iInf / iUnion / iInter over a set Add some lemmas to change variables in `iSup` / `iInf` when the index ranges over a set. There are similar lemmas in the `Equiv` and `Function.Surjective` namespaces but these are over a whole type. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-order 30/0 Mathlib/Data/Set/Lattice.lean,Mathlib/Order/CompleteLattice/Basic.lean 2 3 ['github-actions', 'michelsol', 'urkud'] nobody
1-57359
1 day ago
1-58074
1 day ago
2-41127
2 days
33676 YuvalFilmus
author:YuvalFilmus
feat(Chebyshev/Orthogonality): Chebyshev T polynomials are orthogonal We prove that the Chebyshev T polynomials are orthogonal with respect to `1 / √ (1 - x ^ 2)`. Similarly, one could show that the Chebyshev U polynomials are orthogonal with respect to `√ (1 - x ^ 2)`, which I will do once this PR is approved. More generally, one defines an inner product space on the space of all real polynomials, where the inner product is as defined above. I will be happy to add this to the present or a future PR. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis 173/0 Mathlib.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Chebyshev/Orthogonality.lean 2 7 ['YuvalFilmus', 'github-actions', 'j-loreaux', 'wwylele'] j-loreaux
assignee:j-loreaux
1-51154
1 day ago
1-41078
1 day ago
8-31624
8 days
33435 astrainfinita
author:astrainfinita
feat: algebra automorphisms of monoid algebras --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra
label:t-algebra$
53/3 Mathlib/Algebra/MonoidAlgebra/Basic.lean 1 2 ['github-actions', 'mathlib4-merge-conflict-bot'] kbuzzard
assignee:kbuzzard
1-50299
1 day ago
1-50300
1 day ago
13-11452
13 days
33505 urkud
author:urkud
feat(Analysis/Complex): prove Riemann mapping theorem I'll list dependencies later. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict 1276/53 Mathlib.lean,Mathlib/Analysis/Calculus/Deriv/Inverse.lean,Mathlib/Analysis/Calculus/FDeriv/Equiv.lean,Mathlib/Analysis/Complex/RiemannMapping.lean,Mathlib/Analysis/Complex/UnitDisc/Basic.lean,Mathlib/Analysis/Complex/UnitDisc/Shift.lean,Mathlib/Analysis/SpecialFunctions/Complex/Arg.lean,Mathlib/Analysis/SpecialFunctions/Complex/Log.lean,Mathlib/Tactic/Linter/DirectoryDependency.lean,Mathlib/Topology/Algebra/Group/CompactOpen.lean,Mathlib/Topology/Instances/AddCircle/Defs.lean 11 6 ['SnirBroshi', 'github-actions', 'mathlib4-merge-conflict-bot', 'urkud'] nobody
1-50298
1 day ago
unknown
unknown
33925 harahu
author:harahu
doc(Topology): fix typos Found and fixed by Codex. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology 4/4 Mathlib/Topology/MetricSpace/PartitionOfUnity.lean,Mathlib/Topology/PartitionOfUnity.lean 2 1 ['github-actions'] nobody
1-49024
1 day ago
1-38991
1 day ago
1-38811
1 day
32481 ADedecker
author:ADedecker
feat: add `PolynormableSpace.banach_steinhaus` --- - [x] depends on: #32480 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis delegated 121/24 Mathlib/Analysis/LocallyConvex/AbsConvexOpen.lean,Mathlib/Analysis/LocallyConvex/Barrelled.lean,Mathlib/Analysis/LocallyConvex/WithSeminorms.lean,Mathlib/Analysis/Normed/Operator/BanachSteinhaus.lean 4 4 ['github-actions', 'j-loreaux', 'mathlib-bors', 'mathlib4-dependent-issues-bot'] sgouezel
assignee:sgouezel
1-47810
1 day ago
1-47810
1 day ago
6-2998
6 days
33634 xgenereux
author:xgenereux
feat(ValuationSubring): eq_self_or_eq_top_of_le Using `primeSpectrumEquiv` we get the the corresponding results of `IsLocalRing.primeSpectrum_eq_of_KrullDimLEOne`(see #33607) for valuation subrings. --- - [ ] depends on: #33631 - [ ] depends on: #33612 - [ ] depends on: #33609 - [ ] depends on: #33607 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR large-import 79/18 Mathlib/Algebra/Order/Ring/Ordering/Basic.lean,Mathlib/RingTheory/DedekindDomain/Ideal/Lemmas.lean,Mathlib/RingTheory/Ideal/GoingUp.lean,Mathlib/RingTheory/Ideal/Maps.lean,Mathlib/RingTheory/Ideal/Maximal.lean,Mathlib/RingTheory/Ideal/MinimalPrime/Basic.lean,Mathlib/RingTheory/Ideal/NatInt.lean,Mathlib/RingTheory/Ideal/Prime.lean,Mathlib/RingTheory/Jacobson/Ring.lean,Mathlib/RingTheory/KrullDimension/Basic.lean,Mathlib/RingTheory/KrullDimension/Zero.lean,Mathlib/RingTheory/LocalRing/ResidueField/Fiber.lean,Mathlib/RingTheory/Localization/Ideal.lean,Mathlib/RingTheory/Spectrum/Prime/Basic.lean,Mathlib/RingTheory/Spectrum/Prime/Topology.lean,Mathlib/RingTheory/Valuation/ValuationSubring.lean 16 6 ['alreadydone', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'plp127', 'xgenereux'] nobody
1-43977
1 day ago
unknown
unknown
33814 seewoo5
author:seewoo5
feat(Manifold/MFDeriv): add `MDifferentiable.pow` with FunProp --- - [ ] depends on: #33808 Tag `MDifferentiable.pow` with `fun_prop`. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-differential-geometry blocked-by-other-PR merge-conflict 22/0 Mathlib/Geometry/Manifold/MFDeriv/Basic.lean,Mathlib/Geometry/Manifold/MFDeriv/Defs.lean,Mathlib/Geometry/Manifold/MFDeriv/SpecificFunctions.lean 3 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
1-43853
1 day ago
5-3076
5 days ago
0-7682
2 hours
33857 euprunin
author:euprunin
chore: golf and reduce compilation time --- Trace profiling results (shown if ≥10 ms before or after): * `Finset.prod_ite_mem_eq`: 38 ms before, 16 ms after 🎉 * `Finset.prod_eq_ite`: 82 ms before, 38 ms after 🎉 * `Finset.prod_dite_of_true`: 69 ms before, 30 ms after 🎉 * `Subgroup.forall_mem_sup`: 268 ms before, 51 ms after 🎉 * `Finset.nsmul_piAntidiag`: 277 ms before, 167 ms after 🎉 * `not_mulDissociated`: 642 ms before, 48 ms after 🎉 * `Finset.mem_falling`: 126 ms before, 35 ms after 🎉 * `Finset.image_diag`: 66 ms before, 44 ms after 🎉 * `Finset.biUnion_congr`: 241 ms before, 110 ms after 🎉 * `List.countP_erase`: 197 ms before, 136 ms after 🎉 * `List.triplewise_cons`: 209 ms before, 25 ms after 🎉 * `List.triplewise_append`: 298 ms before, 47 ms after 🎉 * `Nat.primeFactors_gcd`: 77 ms before, 32 ms after 🎉 * `Prod.swap_eq_iff_eq_swap`: 148 ms before, 12 ms after 🎉 * `Set.encard_eq_four`: 1034 ms before, 962 ms after 🎉 * `Set.forall_mem_image2`: 376 ms before, 33 ms after 🎉 * `Set.exists_mem_image2`: 386 ms before, 82 ms after 🎉 * `Set.pairwise_union`: 1219 ms before, 182 ms after 🎉 * `SubMulAction.mem_ofFixingSubgroup_insert_iff`: 310 ms before, 61 ms after 🎉 * `vectorSpan_add_self`: 1727 ms before, 180 ms after 🎉 * `Submodule.mem_sSup_iff_exists_finset`: 1233 ms before, 315 ms after 🎉 * `Matrix.kroneckerMap_single_single`: 436 ms before, 179 ms after 🎉 * `MeasureTheory.integral_biUnion_eq_sum_powerset`: 550 ms before, 247 ms after 🎉 * `NumberField.mixedEmbedding.fundamentalCone.card_isPrincipal_dvd_norm_le`: 945 ms before, 266 ms after 🎉 * `Set.inl_compl_union_inr_compl`: 263 ms before, 167 ms after 🎉 * `Set.ssubset_iff_sdiff_singleton`: 345 ms before, 78 ms after 🎉 * `Sublattice.le_pi`: 398 ms before, 189 ms after 🎉 * `ProbabilityTheory.Kernel.comapRight_compProd_id_prod`: 250 ms before, 145 ms after 🎉 * `Algebra.adjoin_singleton_induction`: 48 ms before, 22 ms after 🎉 * `Ideal.IsPrime.mul_mem_left_iff`: 146 ms before, 141 ms after 🎉 * `Dense.ciSup'`: 277 ms before, 150 ms after 🎉 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 28/34 Mathlib/Algebra/BigOperators/Group/Finset/Basic.lean,Mathlib/Algebra/BigOperators/Group/Finset/Piecewise.lean,Mathlib/Algebra/Group/Subgroup/Lattice.lean,Mathlib/Algebra/Order/Antidiag/Pi.lean,Mathlib/Combinatorics/Additive/Dissociation.lean,Mathlib/Combinatorics/SetFamily/LYM.lean,Mathlib/Data/Finset/Prod.lean,Mathlib/Data/Finset/Union.lean,Mathlib/Data/List/Count.lean,Mathlib/Data/Nat/PrimeFin.lean,Mathlib/Data/Set/Card.lean,Mathlib/Data/Set/NAry.lean,Mathlib/Data/Set/Pairwise/Basic.lean,Mathlib/GroupTheory/GroupAction/SubMulAction/OfFixingSubgroup.lean,Mathlib/LinearAlgebra/AffineSpace/AffineSubspace/Defs.lean,Mathlib/LinearAlgebra/Finsupp/Span.lean,Mathlib/LinearAlgebra/Matrix/Kronecker.lean,Mathlib/MeasureTheory/Integral/Bochner/Set.lean,Mathlib/NumberTheory/NumberField/CanonicalEmbedding/FundamentalCone.lean,Mathlib/Order/BooleanAlgebra/Set.lean,Mathlib/Order/Sublattice.lean,Mathlib/Probability/Kernel/Composition/CompProd.lean,Mathlib/RingTheory/Adjoin/Polynomial.lean,Mathlib/RingTheory/Ideal/Prime.lean,Mathlib/Topology/Order/IsLUB.lean 25 4 ['euprunin', 'github-actions', 'harahu', 'leanprover-radar', 'mathlib4-merge-conflict-bot'] nobody
1-43638
1 day ago
1-28898
1 day ago
3-15326
3 days
33935 mckoen
author:mckoen
feat(CategoryTheory/Arrow): define monoidal structure on the arrow category moves PushoutObjObj, defines monoidal category structure on arrow category, WIP --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP t-category-theory 743/122 Mathlib/CategoryTheory/Comma/Monoidal.lean,Mathlib/CategoryTheory/LiftingProperties/ParametrizedAdjunction.lean,Mathlib/CategoryTheory/Limits/Shapes/Pullback/PullbackObjObj.lean 3 0 [] nobody
1-42147
1 day ago
unknown
unknown
33441 dupuisf
author:dupuisf
feat: add `LawfulInv` class for types with an inverse that behaves like `Ring.inverse` This PR introduces a new typeclass `LawfulInv` for types which have an `Inv` instance that is equal to zero on non-invertible elements. This is meant to replace `Ring.inverse`. The current plan is to do this refactor in several steps: 1. This PR, which only introduces the class and adds instances for matrices and continuous linear maps. 2. Add instances for all C*-algebras, and make `CStarAlgebra` extend this. 3. Deprecate `Ring.inverse`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-algebra
label:t-algebra$
173/22 Mathlib/Algebra/GroupWithZero/Defs.lean,Mathlib/Algebra/GroupWithZero/Invertible.lean,Mathlib/Algebra/GroupWithZero/Units/Basic.lean,Mathlib/LinearAlgebra/Matrix/NonsingularInverse.lean,Mathlib/LinearAlgebra/Matrix/PosDef.lean,Mathlib/RingTheory/DividedPowers/Padic.lean,Mathlib/Topology/Algebra/Module/Equiv.lean 7 30 ['dupuisf', 'eric-wieser', 'github-actions', 'j-loreaux', 'mathlib4-merge-conflict-bot', 'plp127'] nobody
1-41583
1 day ago
1-53086
1 day ago
4-49735
4 days
33491 themathqueen
author:themathqueen
feat(Analysis/InnerProductSpace): linear map is positive iff it equals the sum of rank-one operators ... and equality of nonzero rank-one operators means the elements are colinear. --- - [x] depends on: #33439 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis 59/1 Mathlib/Analysis/InnerProductSpace/LinearMap.lean,Mathlib/Analysis/InnerProductSpace/Positive.lean,Mathlib/Analysis/InnerProductSpace/Symmetric.lean 3 9 ['github-actions', 'j-loreaux', 'mathlib4-dependent-issues-bot', 'themathqueen'] urkud
assignee:urkud
1-41186
1 day ago
1-29507
1 day ago
8-32225
8 days
33882 AntoineChambert-Loir
author:AntoineChambert-Loir
feat(LinearAlgebra/Transvection/SpecialLinearGroup): commutators in the special linear group Over a field, prove the following results : * transvections are conjugate in the general linear group; except in rank 2, they are conjugate in the special linear group. * the special linear group is equal to its commutator subgroup (except when it doesn't, ie, in rank 2 over a field with 2 or 3 elements). --- - [ ] depends on: #33347 - [ ] depends on: #33348 - [ ] depends on: #33387 - [ ] depends on: #33282 - [ ] depends on: #33392 - [ ] depends on: #33402 - [ ] depends on: #33485 - [ ] depends on: #32757 - [ ] depends on: #33560 - [ ] depends on: #33692 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR file-removed 3128/235 Mathlib.lean,Mathlib/GroupTheory/Commutator/Basic.lean,Mathlib/LinearAlgebra/Basis/Fin.lean,Mathlib/LinearAlgebra/Center.lean,Mathlib/LinearAlgebra/Determinant.lean,Mathlib/LinearAlgebra/Dual/Defs.lean,Mathlib/LinearAlgebra/FiniteDimensional/Lemmas.lean,Mathlib/LinearAlgebra/LinearIndependent/Lemmas.lean,Mathlib/LinearAlgebra/SpecialLinearGroup.lean,Mathlib/LinearAlgebra/Transvection.lean,Mathlib/LinearAlgebra/Transvection/Basic.lean,Mathlib/LinearAlgebra/Transvection/Generation.lean,Mathlib/LinearAlgebra/Transvection/SpecialLinearGroup.lean 13 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
1-40634
1 day ago
unknown
unknown
33870 jcommelin
author:jcommelin
feat(Data/Matrix/Cartan): add IsSymm lemmas and simplify IsSimplyLaced proofs This PR adds symmetry theorems for A, D, and E-series Cartan matrices, a DecidablePred instance for IsSimplyLaced, and a lemma reducing simply-laced checks to half the entries for symmetric matrices. The E-series and F₄/G₂ proofs are simplified to use decide. --- - [x] depends on: #33538 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data merge-conflict 37/8 Mathlib/Data/Matrix/Cartan.lean 1 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
1-40253
1 day ago
1-43851
1 day ago
0-13862
3 hours
33631 xgenereux
author:xgenereux
feat(ValuationSubring): simp lemmas for idealOfLE/ofPrime in relation to top/bot simp lemmas for `idealOfLE`/`ofPrime` in the trivial cases of `⊥`, `⊤` . This is my second try at this PR (after I bailed on #33618), sorry about this! --- - [ ] depends on: #33612 - [ ] depends on: #33609 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR 30/0 Mathlib/RingTheory/Valuation/ValuationSubring.lean 1 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
1-38886
1 day ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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 41 ['eric-wieser', 'github-actions', 'jcommelin', 'kckennylau', 'robertmaxton42'] PatrickMassot
assignee:PatrickMassot
1-37760
1 day ago
52-9806
52 days ago
52-9626
52 days
33851 alreadydone
author:alreadydone
chore(Algebra): deprecate `CancelMonoidWithZero` The ring theory library already unbundles classes like `IsDomain`, and it's unusual for the monoid library to use bundled cancellative classes, leading to anti-patterns synthesizing bundled from unbundled like `IsDomain.toCancelMonoidWithZero`. This PR removes `Cancel(Comm)MonoidWithZero` in favor of `[(Comm)MonoidWithZero] [IsCancelMulZero]`. In exchange, `UniqueFactorizationMonoid` and `(Normalized)GCDMonoid` now extend `IsCancelMul`. Inspired by #33832, where generalizing `IsDomain.toCancelMonoidWithZero` to `IsCancelMulZero` led to timeouts. Zulip: https://leanprover.zulipchat.com/#narrow/channel/144837-PR-reviews/topic/.2333851.20deprecate.20CancelMonoidWithZero/near/567433366 TODO: deprecate (Left/Right)CancelSemigroup/Monoid. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
374/381 Mathlib/Algebra/BigOperators/Associated.lean,Mathlib/Algebra/GCDMonoid/Basic.lean,Mathlib/Algebra/GCDMonoid/Finset.lean,Mathlib/Algebra/GCDMonoid/FinsetLemmas.lean,Mathlib/Algebra/GCDMonoid/IntegrallyClosed.lean,Mathlib/Algebra/GCDMonoid/Multiset.lean,Mathlib/Algebra/GroupWithZero/Action/Faithful.lean,Mathlib/Algebra/GroupWithZero/Action/Opposite.lean,Mathlib/Algebra/GroupWithZero/Associated.lean,Mathlib/Algebra/GroupWithZero/Basic.lean,Mathlib/Algebra/GroupWithZero/Defs.lean,Mathlib/Algebra/GroupWithZero/Divisibility.lean,Mathlib/Algebra/GroupWithZero/Idempotent.lean,Mathlib/Algebra/GroupWithZero/InjSurj.lean,Mathlib/Algebra/GroupWithZero/Nat.lean,Mathlib/Algebra/GroupWithZero/Submonoid/Primal.lean,Mathlib/Algebra/GroupWithZero/Torsion.lean,Mathlib/Algebra/GroupWithZero/Units/Basic.lean,Mathlib/Algebra/Order/GroupWithZero/Synonym.lean,Mathlib/Algebra/Order/GroupWithZero/Unbundled/Basic.lean,Mathlib/Algebra/Order/Interval/Set/Instances.lean,Mathlib/Algebra/Order/Monoid/Associated.lean,Mathlib/Algebra/Polynomial/FieldDivision.lean,Mathlib/Algebra/Prime/Defs.lean,Mathlib/Algebra/Prime/Lemmas.lean,Mathlib/Algebra/Regular/Basic.lean,Mathlib/Algebra/Ring/Basic.lean,Mathlib/Algebra/Ring/CharZero.lean,Mathlib/Algebra/Ring/Divisibility/Lemmas.lean,Mathlib/Algebra/Ring/Int/Defs.lean,Mathlib/Algebra/Ring/NonZeroDivisors.lean,Mathlib/Algebra/Ring/PUnit.lean,Mathlib/Algebra/Ring/Rat.lean,Mathlib/Algebra/Ring/Regular.lean,Mathlib/Algebra/Squarefree/Basic.lean,Mathlib/Analysis/Meromorphic/TrailingCoefficient.lean,Mathlib/Analysis/Normed/Field/UnitBall.lean,Mathlib/Combinatorics/Additive/AP/Three/Defs.lean,Mathlib/Data/List/Prime.lean,Mathlib/Data/Matrix/Basic.lean,Mathlib/Data/Matrix/Composition.lean,Mathlib/LinearAlgebra/Eigenspace/Semisimple.lean,Mathlib/RingTheory/ChainOfDivisors.lean,Mathlib/RingTheory/DedekindDomain/Ideal/Basic.lean,Mathlib/RingTheory/DiscreteValuationRing/Basic.lean,Mathlib/RingTheory/IntegralDomain.lean,Mathlib/RingTheory/Multiplicity.lean,Mathlib/RingTheory/Nilpotent/Basic.lean,Mathlib/RingTheory/OreLocalization/OreSet.lean,Mathlib/RingTheory/Polynomial/Content.lean,Mathlib/RingTheory/Polynomial/ContentIdeal.lean,Mathlib/RingTheory/Polynomial/Eisenstein/IsIntegral.lean,Mathlib/RingTheory/Polynomial/Nilpotent.lean,Mathlib/RingTheory/Polynomial/UniqueFactorization.lean,Mathlib/RingTheory/Prime.lean,Mathlib/RingTheory/PrincipalIdealDomain.lean,Mathlib/RingTheory/Radical.lean,Mathlib/RingTheory/RootsOfUnity/PrimitiveRoots.lean,Mathlib/RingTheory/Spectrum/Prime/Polynomial.lean,Mathlib/RingTheory/UniqueFactorizationDomain/Basic.lean,Mathlib/RingTheory/UniqueFactorizationDomain/Defs.lean,Mathlib/RingTheory/UniqueFactorizationDomain/FactorSet.lean,Mathlib/RingTheory/UniqueFactorizationDomain/Finite.lean,Mathlib/RingTheory/UniqueFactorizationDomain/Finsupp.lean,Mathlib/RingTheory/UniqueFactorizationDomain/GCDMonoid.lean,Mathlib/RingTheory/UniqueFactorizationDomain/Ideal.lean,Mathlib/RingTheory/UniqueFactorizationDomain/Multiplicative.lean,Mathlib/RingTheory/UniqueFactorizationDomain/Multiplicity.lean,Mathlib/RingTheory/UniqueFactorizationDomain/NormalizedFactors.lean,Mathlib/SetTheory/Nimber/Field.lean,Mathlib/Tactic/FieldSimp/Lemmas.lean,MathlibTest/grind/panic.lean 72 5 ['alreadydone', 'github-actions', 'leanprover-radar'] nobody
1-37509
1 day ago
1-24941
1 day ago
1-67263
1 day
33766 alreadydone
author:alreadydone
feat(Analysis, Topology): more examples of covering maps involving the complex plane --- - [ ] depends on: #33726 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-topology t-analysis blocked-by-other-PR large-import 311/11 Mathlib/Algebra/Polynomial/Eval/Defs.lean,Mathlib/Algebra/Polynomial/Roots.lean,Mathlib/Analysis/Complex/CoveringMap.lean,Mathlib/Analysis/Complex/OpenMapping.lean,Mathlib/Analysis/SpecialFunctions/Complex/Circle.lean,Mathlib/Data/Nat/Init.lean,Mathlib/FieldTheory/IsAlgClosed/Basic.lean,Mathlib/RingTheory/RootsOfUnity/Basic.lean,Mathlib/Topology/Algebra/GroupWithZero.lean,Mathlib/Topology/Algebra/Polynomial.lean,Mathlib/Topology/Covering/Basic.lean 11 4 ['alreadydone', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
1-36766
1 day ago
unknown
unknown
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` --- - [ ] depends on: #33939 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR t-topology large-import 124/69 Mathlib/Algebra/Order/Monoid/Canonical/Basic.lean,Mathlib/Analysis/Normed/Unbundled/SeminormFromConst.lean,Mathlib/Analysis/Normed/Unbundled/SpectralNorm.lean,Mathlib/Topology/Instances/NNReal/Lemmas.lean,Mathlib/Topology/Instances/Real/Lemmas.lean 5 30 ['YaelDillies', 'github-actions', 'j-loreaux', 'mathlib4-dependent-issues-bot', 'mitchell-horner'] YaelDillies
assignee:YaelDillies
1-32199
1 day ago
1-32200
1 day ago
38-61422
38 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 66/1 Mathlib/Topology/Algebra/Module/ClosedSubmodule.lean 1 4 ['github-actions', 'j-loreaux', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] fpvandoorn
assignee:fpvandoorn
1-31865
1 day ago
1-21538
1 day ago
77-63270
77 days
32777 madvorak
author:madvorak
doc: Contributing moved to Contributing --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 54/56 .github/CONTRIBUTING.md,README.md 2 2 ['github-actions'] Vierkantor
assignee:Vierkantor
1-31240
1 day ago
34-4536
34 days ago
34-4356
34 days
33118 thomaskwaring
author:thomaskwaring
feat(Combinatorics/SimpleGraph/Acyclic): every graph has a spanning forest. We show that every graph has a spanning forest: defined to be an acyclic subgraph with the same reachability relation as the larger graph. As a special case, every connected graph has a spanning tree. --- Each of these results (spanning forest & spanning tree) are proved in two versions: a general case where the forest / tree is found by extending a given acyclic subgraph, and the special case where that subgraph is empty. - [ ] depends on: #32043 new-contributor t-combinatorics 29/5 Mathlib/Combinatorics/SimpleGraph/Acyclic.lean 1 6 ['SnirBroshi', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'thomaskwaring', 'vlad902'] b-mehta
assignee:b-mehta
1-31238
1 day ago
11-27941
11 days ago
12-13936
12 days
33253 SnirBroshi
author:SnirBroshi
feat(Combinatorics/SimpleGraph/Clique): avoid `Fintype`/`Finite` assumptions where possible Also prove `G.cliqueNum ≤ G.chromaticNumber` without any finiteness assumptions. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics 39/40 Mathlib/Combinatorics/SimpleGraph/Clique.lean,Mathlib/Combinatorics/SimpleGraph/Coloring.lean 2 1 ['github-actions'] kmill
assignee:kmill
1-31237
1 day ago
21-75111
21 days ago
21-74931
21 days
33288 vihdzp
author:vihdzp
chore(Combinatorics/SimpleGraph/Paths): review API This PR does the following: - Add `grind` annotations. - Rename theorems `X_isY` to the more idiomatic `isY_X`. - Remove many redundant namespaces. - Golf accordingly. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics 154/122 Mathlib/Combinatorics/SimpleGraph/Acyclic.lean,Mathlib/Combinatorics/SimpleGraph/Connectivity/Connected.lean,Mathlib/Combinatorics/SimpleGraph/Matching.lean,Mathlib/Combinatorics/SimpleGraph/Metric.lean,Mathlib/Combinatorics/SimpleGraph/Paths.lean,Mathlib/Combinatorics/SimpleGraph/Walks/Maps.lean 6 2 ['github-actions', 'mathlib4-merge-conflict-bot'] b-mehta
assignee:b-mehta
1-31236
1 day ago
7-37786
7 days ago
10-63297
10 days
33292 SnirBroshi
author:SnirBroshi
feat(Combinatorics/SimpleGraph/LineGraph): lift copies/isomorphisms to line-graph --- Non-injective homomorphisms (`G →g G'`) cannot be lifted to a homomorphism on line-graphs (`G.lineGraph →g G'.lineGraph`) because e.g. `∀ k > 1` there is a homomorphism from `pathGraph k` to `G'` iff `G'` has an edge, and `∀ n > 0, (pathGraph (n + 1)).lineGraph ≃ pathGraph n`, but there is no homomorphism from `pathGraph k` to `pathGraph 1` because it has no edges. So for `G := pathGraph 3` and `G' := pathGraph 2` there is a `G →g G'` but no `G.lineGraph →g G'.lineGraph`. But we can lift `Copy`/`Embedding`/`Iso`. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-combinatorics 47/4 Mathlib/Combinatorics/SimpleGraph/LineGraph.lean,Mathlib/Data/Sym/Sym2.lean 2 1 ['github-actions'] b-mehta
assignee:b-mehta
1-31235
1 day ago
19-11472
19 days ago
20-33194
20 days
33335 YaelDillies
author:YaelDillies
feat(Combinatorics/SimpleGraph): more about two-reachability --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics 51/51 Mathlib/Combinatorics/SimpleGraph/Connectivity/Connected.lean,Mathlib/Combinatorics/SimpleGraph/Connectivity/EdgeConnectivity.lean,Mathlib/Combinatorics/SimpleGraph/DeleteEdges.lean 3 3 ['SnirBroshi', 'YaelDillies', 'github-actions'] kmill
assignee:kmill
1-31234
1 day ago
16-461
16 days ago
16-281
16 days
33347 AntoineChambert-Loir
author:AntoineChambert-Loir
feat(LinearAlgebra/Transvection/Basic): define dilatransvections Define `LinearEquiv.dilatransvections`. These are linear equivalences whose associated linear map is a transvection. This definition has the interest of being usable without any assumption on the base ring. Over a division ring, they correspond exactly to those linear equivalences `e` such that `e - LinearMap.id` has rank at most one. They (will) appear in Dieudonné's theorem that describes the generation of elements of the general linear group as products of several transvections and one additional dilatransvection. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
204/32 Mathlib/LinearAlgebra/Transvection.lean 1 15 ['AntoineChambert-Loir', 'eric-wieser', 'github-actions', 'mathlib4-merge-conflict-bot'] riccardobrasca
assignee:riccardobrasca
1-31233
1 day ago
4-72418
4 days ago
15-68727
15 days
33360 joelriou
author:joelriou
feat(Algebra/Homology): functoriality of `extMk` with respect to the injective resolution The dual statement for projective resolutions is also obtained. --- - [x] depends on: #33358 - [x] depends on: #32816 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory 206/7 Mathlib/Algebra/Homology/HomotopyCategory/HomComplexSingle.lean,Mathlib/CategoryTheory/Abelian/Injective/Ext.lean,Mathlib/CategoryTheory/Abelian/Injective/Extend.lean,Mathlib/CategoryTheory/Abelian/Projective/Ext.lean,Mathlib/CategoryTheory/Abelian/Projective/Extend.lean,Mathlib/CategoryTheory/Preadditive/Injective/Resolution.lean,Mathlib/CategoryTheory/Preadditive/Projective/Resolution.lean 7 4 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] adamtopaz
assignee:adamtopaz
1-31232
1 day ago
4-50977
4 days ago
4-50797
4 days
33431 gululu996-ui
author:gululu996-ui
feat(Combinatorics/SimpleGraph/Bipartite): characterize bipartite simplegraphs by even cycles Add the classical characterization of bipartite simple graphs: a simple graph is bipartite if and only if every cycle has even length. Previously, mathlib has the definition of `IsBipartite` for `SimpleGraph` and various lemmas about bipartite graphs, but it does not provide this equivalence in a single theorem, so users have to reprove or reassemble it from existing results. Prove the forward direction by showing a 2-coloring alternates along any walk, so every cycle must have even length. Prove the converse by showing that if an odd cycle exists then no bipartition is possible, hence if all cycles are even the graph admits a bipartition. new-contributor t-combinatorics 185/1 Mathlib/Combinatorics/SimpleGraph/Bipartite.lean 1 3 ['NickAdfor', 'github-actions'] kmill
assignee:kmill
1-31232
1 day ago
10-73380
10 days ago
10-73200
10 days
33527 SnirBroshi
author:SnirBroshi
feat(Combinatorics/SimpleGraph/Connectivity/Subgraph): `w.toSubgraph ≤ G' ↔ w.edgeSet ⊆ G'.edgeSet` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics 9/1 Mathlib/Combinatorics/SimpleGraph/Connectivity/Subgraph.lean 1 4 ['Rida-Hamadani', 'SnirBroshi', 'github-actions'] kmill
assignee:kmill
1-31231
1 day ago
11-46961
11 days ago
11-46781
11 days
33804 tb65536
author:tb65536
feat(RingTheory/Localization/Ideal): `map` distributes over `inf` This PR proves that mapping ideals to the localization distributes over finite intersections, following the design of the analogous statements for `Ideal.radical`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-ring-theory t-algebra
label:t-algebra$
24/0 Mathlib/RingTheory/Localization/Ideal.lean 1 6 ['erdOne', 'github-actions', 'plp127', 'tb65536'] mattrobball
assignee:mattrobball
1-31228
1 day ago
4-42150
4 days ago
5-36908
5 days
33818 JohnnyTeutonic
author:JohnnyTeutonic
feat(Algebra/Lie/Classical): finrank of sl(n) equals n² - 1 Proves `finrank R (sl n R) = Fintype.card n ^ 2 - 1` using rank-nullity and `Matrix.trace_surjective`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
10/2 Mathlib/Algebra/Lie/Classical.lean 1 8 ['JohnnyTeutonic', 'github-actions', 'themathqueen'] alreadydone
assignee:alreadydone
1-31227
1 day ago
4-62817
4 days ago
4-70915
4 days
33825 euprunin
author:euprunin
chore: golf using `grind` --- The goal of this golfing PR is to decrease the number of times lemmas are called explicitly (replacing calls to lemmas with calls to tactics). Any decrease in compilation time is a welcome side effect, although it is not a primary objective. Trace profiling results (shown if ≥10 ms before or after): * `Finset.prod_insert_of_eq_one_if_notMem`: <10 ms before, 23 ms after * `Finset.sym2_mono`: <10 ms before, 64 ms after * `Finsupp.support_onFinset_subset`: <10 ms before, 14 ms after * `Disjoint.ne_top_of_ne_bot`: <10 ms before, <10 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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 4/10 Mathlib/Algebra/BigOperators/Group/Finset/Basic.lean,Mathlib/Data/Finset/Sym.lean,Mathlib/Data/Finsupp/Defs.lean,Mathlib/Order/Disjoint.lean 4 1 ['github-actions'] JovanGerb
assignee:JovanGerb
1-31225
1 day ago
4-42529
4 days ago
4-42349
4 days
33132 BoltonBailey
author:BoltonBailey
feat(Computability): Single-tape TM complexity Currently, time complexity in mathlib is defined in terms of (a kind of) multi-tape Turing machine [Turing.FinTM2](https://leanprover-community.github.io/mathlib4_docs/Mathlib/Computability/TMComputable.html#Turing.FinTM2). This (currently Draft) PR develops time complexity in terms of Single-Tape Turing Machines. There are a few reasons to do this: * Having definitions of time complexity for both single-tape and multi-tape TMs is a prerequisite to prove theorems relating these definitions of complexity (in particular, the theorem that the definition of polynomial time computability is equivalent between these notions). * The Multi-tape "TM2" definition seems to be based on "Wang B-Machines" ([wiki](https://en.wikipedia.org/wiki/Wang_B-machine)) which involves both a program of function labels, as well as a set of states. * I think it's a bit more common to see a simpler presentation of single-tape ([and multitape](https://en.wikipedia.org/wiki/Multitape_Turing_machine)) Turing machines which only provides a set of states. * It seems to me that the B-Machine-like definition makes it a bit complicated to make progress. For example, if I want to compose Turing Machines, then I have to be able to construct a new program and state set, which involves mapping the [Turing.TM2.Stmt](https://leanprover-community.github.io/mathlib4_docs/Mathlib/Computability/TuringMachine.html#Turing.TM2.Stmt) type to the sum type of the tapes. I have to do something similar for single-tape TMs, but the Stmt type is less complicated, so this is less involved. * If we want to continue on and define space complexity, it seems convenient to have only a single tape, so that we don't have to do lots of reasoning over summations. ## Models Note [this](https://www.youtube.com/live/pa5mURjUNFI) (h/t Ching-Tsun Chou) talk which discusses "dying in the details" of formalizing complexity theory. I guess the point is that there are a lot of details to choose about the model, which I think is true even for single tape Turing machines, which can make things easier or harder. * Do we allow arbitrary finite tape alphabets, or force all encodings to be Bool? * What is the alphabet of the tape? Is it the alphabet of the input, with an inhabited instance for blank elements (how, then, do we know what the input is). Is it an option type? * Does a single TM tape "statement"/action consist of both writing and moving, or only one or the other? * Do we allow no movement, or must every step involve movement? * Do we require that to be considered to have computed a function, the Turing Machine head must end at the LHS of the tape? * Should we model state transition systems as functions `State -> Option State`, or `State -> `Sum State ReturnType` * Do we formalize multiple of these, and prove equivalences back and forth? ## Other Preliminary Changes? ### Refactor state transition The initial segment of PostTuringMachine.lean seems to have a few definitions about general notions of reachability that could be refactored into a new file. It also feels like TMComputable.lean could use this API. - [ ] depends on: #33291 ### Refactor Concept of "Machine/Automata" There are a number of constructs that have the following structure * A class of objects that broadly represent classes of computable (perhaps partial) functions, with individual functions implemented by individual machines within the class * A machine can have multiple "configurations" which correspond to states of input feed, external tapes and stacks, and internal state. * To compute the function, there is a map from terms of the input type to configurations * There is then a transition function which maps configurations to other configurations, until eventually there is a final configuration which maps to a return type (I have thought it might be better to have the state transitions return a sum type rather than an option to represent this). I am thinking of a few things that could fall under a refactor like this: * DFA * NFA (with states as subsets of states) * epsNFA * TMs (single tape, multi tape, stack, the B-machine things) ### Directory Structure Rather than having multiple files that start with "TM" or have "TuringMachine" in them, perhaps we could put these in one directory? ### Naming of TM0 TM1 TM2 These names unfortunately do not provide the reader with information about what model is being used, so it is somewhat akin to a primed definition. I think I would prefer more descriptive names. ### Namespacing Another note: The naming of things like [Turing.TM2Computable](https://leanprover-community.github.io/mathlib4_docs/Mathlib/Computability/TMComputable.html#Turing.TM2Computable), [Turing.TM2OutputsInTime](https://leanprover-community.github.io/mathlib4_docs/Mathlib/Computability/TMComputable.html#Turing.TM2OutputsInTime) and [Turing.TM2ComputableInTime](https://leanprover-community.github.io/mathlib4_docs/Mathlib/Computability/TMComputable.html#Turing.TM2ComputableInTime) feels a bit unfortunate to me because * These definitions are based on [Turing.FinTM2](https://leanprover-community.github.io/mathlib4_docs/Mathlib/Computability/TMComputable.html#Turing.FinTM2). There is not a "TM2" itself, I guess because it would be weird to allow TMs with infinite alphabets or states. I don't know if the authors originally wanted to allow room for this, but it feels like "FinTM2" should be extending some "TM2" with finiteness. * Because there could be multiple notions of computability-in-time for different machines, the namespace should be Turing.FinTM2.OutputsInTime so that I can use dot-notation. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-computability WIP blocked-by-other-PR 1480/0 Mathlib/Computability/BinEncoding.lean,Mathlib/Computability/EncodingTo.lean,Mathlib/Computability/SingleTapeBinTMComputable.lean,Mathlib/Computability/SingleTapeTMComputable.lean 4 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
1-30738
1 day ago
unknown
unknown
33934 tb65536
author:tb65536
chore(Algebra/Polynomial/Splits): deprecate `Splits.splits` and `splits_iff_splits` After the big refactor of `Polynomial.Splits`, there were two clunky lemmas without good names. This PR deprecates them. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
45/38 Mathlib/Algebra/Polynomial/Splits.lean,Mathlib/FieldTheory/AbelRuffini.lean,Mathlib/FieldTheory/IsAlgClosed/Basic.lean,Mathlib/FieldTheory/IsSepClosed.lean,Mathlib/FieldTheory/Normal/Defs.lean,Mathlib/FieldTheory/SeparableDegree.lean 6 1 ['github-actions'] nobody
1-30396
1 day ago
1-30396
1 day ago
1-30216
1 day
33542 yuanyi-350
author:yuanyi-350
feat(integral): Error Estimation for the Rectangle Rule in Numerical Integration --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-analysis 184/0 Mathlib.lean,Mathlib/Analysis/Calculus/ContDiff/Defs.lean,Mathlib/Analysis/Calculus/Midpoint.lean 3 4 ['github-actions', 'tb65536'] ADedecker
assignee:ADedecker
1-25292
1 day ago
1-40475
1 day ago
4-71666
4 days
33943 urkud
author:urkud
feat(Asymptotics/TVS): add more lemmas I need these to generalize some lemmas about derivatives. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) feat(Asymptotics/TVS): add more lemmas t-analysis 98/0 Mathlib/Analysis/Asymptotics/TVS.lean 1 1 ['github-actions'] nobody
1-22561
1 day ago
1-17213
1 day ago
1-17033
1 day
33582 urkud
author:urkud
feat(ContDiffHolder/Moreira): define $C^{k+(α)}$ maps From https://github.com/urkud/SardMoreira --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis 279/0 Mathlib.lean,Mathlib/Analysis/Calculus/ContDiffHolder/Pointwise.lean,Mathlib/Analysis/SpecialFunctions/Pow/Asymptotics.lean 3 10 ['ADedecker', 'github-actions', 'urkud'] ADedecker
assignee:ADedecker
1-22424
1 day ago
1-14163
1 day ago
8-9016
8 days
33206 lua-vr
author:lua-vr
feat(Integral.Bochner.Set): add `tendsto_setIntegral_of_monotone₀` Adds the lemma `tendsto_setIntegral_of_monotone₀`, a version of `tendsto_setIntegral_of_monotone` requiring only `AEMeasurableSet` in the hypothesis. The previous version is redefined as a specialization. Also renames `integral_union_ae` to `setIntegral_union₀` for consistency with the rest of the library (it matches the existing `setIntegral_union`). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-measure-probability 27/13 Mathlib/MeasureTheory/Integral/Bochner/Set.lean 1 4 ['ADedecker', 'github-actions', 'mathlib4-merge-conflict-bot', 'mcdoll'] RemyDegenne
assignee:RemyDegenne
1-20209
1 day ago
1-60660
1 day ago
21-8588
21 days
33876 joelriou
author:joelriou
feat(Order): `WithBotTop` and the extended integers This files defines an abbreviation `WithBotTop ι` for `WithBot (WithTop ι)`. We also introduce an abbreviation `EInt` for `WithBotTop ℤ`. Kevin Buzzard is made a coauthor of the file because it is very similar to `Data.EReal.Basic`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-data
label:t-algebra$
79/0 Mathlib.lean,Mathlib/Order/WithBotTop.lean 2 8 ['ADedecker', 'github-actions', 'joelriou', 'vihdzp'] nobody
1-19170
1 day ago
1-69444
1 day ago
2-26791
2 days
33884 vihdzp
author:vihdzp
chore(Order/Hom/BoundedLattice): remove `initialize_simps_projections` --- Follow-up to #30378, see [this comment](https://github.com/leanprover-community/mathlib4/pull/30378#issuecomment-3453031006). [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order 6/11 Mathlib/Order/Hom/BoundedLattice.lean,Mathlib/Order/Hom/WithTopBot.lean 2 1 ['github-actions'] nobody
1-18600
1 day ago
1-11970
1 day ago
1-11790
1 day
33948 anivegesana
author:anivegesana
feat(Analysis/Normed/Algebra): matrix exponential of nilpotent matrix Where the matrix exponential and nilpotent elements are defined, both the matrix exponential and the nilpotent element exponential. I had to add a different theorem for normed space exponential and the matrix exponential since the right instances wouldn't be synthesized. Help with golfing would be appreciated. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-analysis 34/0 Mathlib/Analysis/Normed/Algebra/Exponential.lean,Mathlib/Analysis/Normed/Algebra/MatrixExponential.lean 2 1 ['github-actions'] nobody
1-16950
1 day ago
unknown
unknown
33270 vihdzp
author:vihdzp
chore(Order/Disjoint): use `to_dual` --- - [x] depends on: #33268 I'm unsure about the dualized names for some of the new theorems, suggestions welcome. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order awaiting-author 30/87 Mathlib/Order/Disjoint.lean 1 4 ['JovanGerb', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
1-16429
1 day ago
21-12663
21 days ago
0-4
4 seconds
15355 adomani
author:adomani
feat: MiM PR report --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP 153/0 .github/workflows/monthly_pr_report.yaml,scripts/find_labels.sh 2 11 ['YaelDillies', 'adomani', 'github-actions', 'vihdzp'] nobody
1-15390
1 day ago
unknown
unknown
33119 euprunin
author:euprunin
chore: golf using `grind` --- **Note.** Note that although this PR contains substantial golfing, some of the changes lead to slower compilation times, so there is a clear trade-off to consider. Reviewer input is welcome. --- The goal of this golfing PR is to decrease the number of times lemmas are called explicitly (replacing calls to lemmas with calls to tactics). Any decrease in compilation time is a welcome side effect, although it is not a primary objective. Trace profiling results (shown if ≥10 ms before or after): * `prime_pow_iff`: 14 ms before, 62 ms after * `Turing.BlankRel.trans`: <10 ms before, 126 ms after * `Finset.eq_singleton_iff_nonempty_unique_mem`: <10 ms before, 56 ms after * `Orientation.inner_eq_zero_iff_eq_zero_or_eq_smul_rotation_pi_div_two`: 90 ms before, 55 ms after 🎉 * `Equiv.swap_bijOn_self`: 11 ms before, 83 ms after * `Equiv.swap_bijOn_exchange`: <10 ms before, 100 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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author 5/47 Mathlib/Algebra/GroupWithZero/Associated.lean,Mathlib/Computability/Tape.lean,Mathlib/Geometry/Euclidean/Angle/Oriented/Rotation.lean,Mathlib/Logic/Equiv/Set.lean 4 10 ['JovanGerb', 'euprunin', 'github-actions', 'j-loreaux', 'mathlib4-merge-conflict-bot'] nobody
1-12767
1 day ago
23-62009
23 days ago
2-22480
2 days
33689 BoltonBailey
author:BoltonBailey
refactor(Probability): make PMF return NNReal This PR refactors the PMF FunLike instance to return an NNReal rather than an ENNReal. Potentially this could make algebraic manipulation of these return values easier. There are other ways this could be done. In particular, the type `PMF a` is apparently just the type of probability measures over the discrete measure space on the type a. So perhaps we could define `PMF` directly in this way to unify the APIs. This is currently heavily LLM generated and unaudited, so this is a WIP. Zulip discussions: - [#new members > Why is the codomain of PMF in mathlib ENNReal and not NNReal @ 💬](https://leanprover.zulipchat.com/#narrow/channel/113489-new-members/topic/Why.20is.20the.20codomain.20of.20PMF.20in.20mathlib.20ENNReal.20and.20not.20NNReal/near/526572449) - [#new members > Performing arithmetic with ENNReals @ 💬](https://leanprover.zulipchat.com/#narrow/channel/113489-new-members/topic/Performing.20arithmetic.20with.20ENNReals/near/525936290) - [#Is there code for X? > Statistical distance for `PMF`s? @ 💬](https://leanprover.zulipchat.com/#narrow/channel/217875-Is-there-code-for-X.3F/topic/Statistical.20distance.20for.20.60PMF.60s.3F/near/525234190) - [#mathlib4 > PMF Refactor: FunLike vs Definition Change](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/PMF.20Refactor.3A.20FunLike.20vs.20Definition.20Change/with/567771586) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-measure-probability WIP 323/111 Mathlib/Probability/ProbabilityMassFunction/Basic.lean,Mathlib/Probability/ProbabilityMassFunction/Monad.lean 2 1 ['github-actions'] nobody
1-9772
1 day ago
unknown
unknown
26986 WangYiran01
author:WangYiran01
feat(Partition): add bijection for partitions with max part ≤ r 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. Contributed by Yiran Wang. awaiting-author t-combinatorics new-contributor 92/0 Mathlib/Combinatorics/Enumerative/Partition/Basic.lean,Mathlib/Data/Multiset/Lattice.lean 2 19 ['WangYiran01', 'github-actions', 'jcommelin', 'kckennylau', 'kim-em', 'mathlib4-merge-conflict-bot'] b-mehta
assignee:b-mehta
1-7379
1 day ago
7-1341
7 days ago
120-65801
120 days
33894 vihdzp
author:vihdzp
chore: move `Archimedean` to a new `Defs` file I've also moved the most basic theorems (`exists_nat_lt`, etc.) to this file. This greatly decreases the imports needed to use these classes. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
119/66 Mathlib.lean,Mathlib/Algebra/Order/Archimedean/Basic.lean,Mathlib/Algebra/Order/Archimedean/Defs.lean,Mathlib/Data/Real/Archimedean.lean 4 2 ['github-actions', 'vihdzp'] nobody
1-7276
1 day ago
1-10875
1 day ago
1-10695
1 day
33788 harahu
author:harahu
chore(Algebra): move `LinearMap.ker_restrictScalars` Resolve an old TODO by moving `LinearMap.ker_restrictScalars` to a location in `Mathlib/Algebra/Module/Submodule`. The TODO referenced lemmas in plural, but only `LinearMap.ker_restrictScalars` seemed to fit. I assume any other lemmas might already have been moved at an earlier point. --- Notes for reviewers: - The new location in `Mathlib/Algebra/Module/Submodule/Ker.lean` was chosen somewhat arbitrarily in favor of `Mathlib/Algebra/Module/Submodule/RestrictScalars.lean`. Please consider whether `Ker.lean` is the optimal location for this lemma. - I haven't moved content in mathlib before – do I need to add a deprecation alias in the original file, or is the way I've done it fine? [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
14/17 Mathlib/Algebra/Algebra/Basic.lean,Mathlib/Algebra/Module/Submodule/Ker.lean 2 4 ['github-actions', 'mathlib4-merge-conflict-bot', 'mcdoll', 'tb65536'] nobody
1-7209
1 day ago
1-4675
1 day ago
5-24376
5 days
33726 alreadydone
author:alreadydone
feat(Analysis): (complex) polynomials as branched coverings originally proposed by @urkud in #33425 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-topology t-analysis 129/1 Mathlib/Algebra/Polynomial/Roots.lean,Mathlib/Analysis/Complex/CoveringMap.lean,Mathlib/Topology/Algebra/Polynomial.lean,Mathlib/Topology/Covering/Basic.lean 4 10 ['alreadydone', 'github-actions', 'j-loreaux', 'mathlib4-merge-conflict-bot'] nobody
1-5982
1 day ago
1-5982
1 day ago
6-76093
6 days
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 - [x] depends on: #30348 - [ ] depends on: #30582 - [x] depends on: #31551 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) --- *This PR continues the work from #24430.* *Original PR: https://github.com/leanprover-community/mathlib4/pull/24430* WIP blocked-by-other-PR t-measure-probability merge-conflict 1340/5 Mathlib.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/UniformSpace/AbstractCompletion.lean,docs/1000.yaml 11 13 ['github-actions', 'grunweg', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
1-5967
1 day ago
unknown
unknown
33388 plby
author:plby
doc(docs/100.yaml): add recently-proven theorems Two theorems from Freek Wiedijk's list of 100 theorems are currently in a Mathlib PR in progress. Five theorems from the list have been auto-formalized by Aristotle from Harmonic, and their solutions are hosted elsewhere. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict new-contributor awaiting-author 43/1 docs/100.yaml,docs/1000.yaml 2 26 ['Ruben-VandeVelde', 'github-actions', 'jcommelin', 'jsm28', 'mathlib4-merge-conflict-bot', 'mo271', 'ocfnash', 'plby', 'wwylele'] jcommelin, kim-em, ocfnash
assignee:kim-em assignee:jcommelin assignee:ocfnash
1-4233
1 day ago
7-70272
7 days ago
6-74167
6 days
33765 JovanGerb
author:JovanGerb
feat(Order/CompleteLattice/Defs): `to_dual` for `CompleteSemilattice`s This PR uses `to_dual` for `CompleteSemilatticeSup` and `CompleteSemilatticeInf`. These will need to be refactored/deprecated in the future, but I think it makes sense to make the code smaller (using `to_dual`) before such a refactor. --- - [ ] depends on: #33760 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR large-import t-order 157/360 Mathlib/Order/Bounds/Basic.lean,Mathlib/Order/Bounds/Defs.lean,Mathlib/Order/CompleteLattice/Defs.lean,Mathlib/Order/Interval/Set/Defs.lean,Mathlib/Tactic/Translate/ToDual.lean 5 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'vihdzp'] nobody
1-3550
1 day ago
unknown
unknown
33506 Rida-Hamadani
author:Rida-Hamadani
feat(SimpleGraph): construct a cycle of two distinct paths with same start and end --- - [ ] depends on: #33249 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR t-combinatorics 263/1 Mathlib/Combinatorics/SimpleGraph/Connectivity/WalkDecomp.lean,Mathlib/Combinatorics/SimpleGraph/Paths.lean,Mathlib/Combinatorics/SimpleGraph/Walks/Operations.lean,Mathlib/Combinatorics/SimpleGraph/Walks/Subwalks.lean,Mathlib/Combinatorics/SimpleGraph/Walks/Traversal.lean,Mathlib/Data/List/Basic.lean,Mathlib/Data/List/Infix.lean 7 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
1-3515
1 day ago
12-14252
12 days ago
0-5
5 seconds
32891 felixpernegger
author:felixpernegger
feat(Topology/EMetricSpace): Introduction of ```Weak(Pseudo)EMetricSpace``` This PR introduces Weak(Pseudo)EMetric spaces, some basic properties and the fact that the One-Point Compactification of a Weak(Pseudo)EMetricSpace again has a Weak(Pseudo)EMetricSpace structure. This is inspired by discussion at [this](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/EMetricSpace.20is.20broken/near/530540916) and based on #27756. In short, types like ```ENNReal``` and ```ENat``` have a very "metric-like" structure, but are not yet a ```WeakPseudoEMetricSpace``` (which is the weakest form of a metric-like structure in mathlib). Therefore, the class```WeakEMetricSpace``` could be used to make more definitions applicable to ```ENNReal```, for instance EVartiationOn ([this](https://leanprover-community.github.io/mathlib4_docs/Mathlib/Topology/EMetricSpace/BoundedVariation.html#eVariationOn)). As of now, this PR is still missing important properties like products and induced (and therefore subtypes) of ```Weak(Pseudo)EMetricSpace```'s and instances ```ENNReal``` and ```ENat``` (which should be rather easy however with the one-point compactification property). new-contributor t-topology 470/10 Mathlib.lean,Mathlib/Topology/EMetricSpace/Defs.lean,Mathlib/Topology/EMetricSpace/Weak.lean 3 4 ['felixpernegger', 'github-actions', 'mathlib4-merge-conflict-bot', 'plp127'] j-loreaux
assignee:j-loreaux
1-3479
1 day ago
4-56139
4 days ago
7-14039
7 days
33767 Whysoserioushah
author:Whysoserioushah
chore(RingTheory/Morita/Matrix): Finish the morita equivalence between matrix ring and the ring itself --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-ring-theory large-import 79/1 Mathlib/RingTheory/Morita/Matrix.lean 1 12 ['Whysoserioushah', 'eric-wieser', 'github-actions'] erdOne
assignee:erdOne
1-3339
1 day ago
6-15827
6 days ago
6-50535
6 days
33636 mcdoll
author:mcdoll
feat(Analysis/Distribution): the Laplacian on Schwartz functions We introduce a notation type-class for the Laplacian, change the definition of `InnerProductSpace.laplacian` to `Laplacian.laplacian` and define the Laplacian using the sum of second derivatives on Schwartz functions. We define an abstract Laplacian for any space with `LineDeriv` in order to avoid duplication for other function spaces (in particular, this will be reused for the tempered distribution Laplacian). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-analysis 199/12 Mathlib.lean,Mathlib/Analysis/Distribution/DerivNotation.lean,Mathlib/Analysis/Distribution/Laplacian.lean,Mathlib/Analysis/Distribution/SchwartzSpace.lean,Mathlib/Analysis/InnerProductSpace/Harmonic/Basic.lean,Mathlib/Analysis/InnerProductSpace/Laplacian.lean 6 8 ['github-actions', 'j-loreaux', 'mcdoll', 'sgouezel'] urkud
assignee:urkud
1-643
1 day ago
1-643
1 day ago
6-13505
6 days
33087 joelriou
author:joelriou
feat(AlgebraicTopology): the cofibrant resolution functor (up to homotopy) Let `C` be a model category. By using the right homotopy relation, we introduce the homotopy category `CofibrantObject.π C` of cofibrant objects in `C`, and we define a cofibrant resolution functor `CofibrantObject.π.resolution : C ⥤ CofibrantObject.π C`. --- - [x] depends on: #33084 - [x] depends on: #33085 - [x] depends on: #33086 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebraic-topology 220/0 Mathlib.lean,Mathlib/AlgebraicTopology/ModelCategory/CofibrantObjectHomotopy.lean 2 4 ['github-actions', 'joelriou', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
0-85183
23 hours ago
0-84269
23 hours ago
0-84089
23 hours
33606 ScottCarnahan
author:ScottCarnahan
feat(Algebra/Lie): basics of loop algebras This PR introduces the Lie algebra of polynomial loops in a base Lie algebra, together with the 2-cocycle induced by a symmetric invariant bilinear form on the base Lie algebra. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
201/1 Mathlib.lean,Mathlib/Algebra/Lie/BaseChange.lean,Mathlib/Algebra/Lie/Extension.lean,Mathlib/Algebra/Lie/Loop.lean 4 1 ['github-actions'] ocfnash
assignee:ocfnash
0-84367
23 hours ago
2-36786
2 days ago
6-52506
6 days
33939 mitchell-horner
author:mitchell-horner
chore(Analysis/Normed): redefine `seminormFromConst'` without `choose` Redefine `seminormFromConst'` using `iInf` instead of `choose`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 136/94 Mathlib.lean,Mathlib/Analysis/Normed/Unbundled/SeminormFromConst.lean,Mathlib/Analysis/Normed/Unbundled/SpectralNorm.lean,Mathlib/Topology/Instances/NNReal/Lemmas.lean,Mathlib/Topology/Instances/Real/Lemmas.lean,Mathlib/Topology/Instances/Real/Periodic.lean 6 14 ['github-actions', 'mitchell-horner', 'vihdzp'] nobody
0-81918
22 hours ago
0-84502
23 hours ago
1-10203
1 day
33954 or4nge19
author:or4nge19
feat(CategoryTheory/Abelian): add Filtration API Filtered objects in an abelian category (Deligne, *Théorie de Hodge II*, §1.1). Opposed filtrations (Deligne, *Théorie de Hodge II*, §1.2.1–§1.2.3). Induced filtrations on graded pieces (Deligne, *Théorie de Hodge II*, §1.2.1). Co-authored-by: Jonathan Washburn --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-category-theory 565/0 Mathlib.lean,Mathlib/CategoryTheory/Filtration/Basic.lean,Mathlib/CategoryTheory/Filtration/InducedOnGr.lean,Mathlib/CategoryTheory/Filtration/Opposed.lean 4 2 ['github-actions', 'joelriou'] nobody
0-81703
22 hours ago
unknown
unknown
33952 vihdzp
author:vihdzp
chore(Order/FixedPoints): use `where` notation This also avoids constructing auxiliary `CompleteSemilatticeInf` and `CompleteSemilatticeSup` instances. These are meant exclusively to build a `CompleteLattice` from one without the other; this isn't what's happening here. See [Zulip](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Ditch.20CompleteSemilatticeSup/near/567390440). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order 27/36 Mathlib/Order/FixedPoints.lean 1 2 ['eric-wieser', 'github-actions'] nobody
0-81325
22 hours ago
1-2057
1 day ago
1-1877
1 day
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? [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) delegated t-meta 55/14 Mathlib/Tactic/Abel.lean,Mathlib/Tactic/FieldSimp.lean,Mathlib/Tactic/Ring/RingNF.lean,Mathlib/Util/AtomM/Recurse.lean,MathlibTest/FieldSimp.lean 5 29 ['FLDutchmann', 'JovanGerb', 'Vierkantor', 'github-actions', 'grunweg', 'leanprover-radar', 'mathlib-bors'] alexjbest
assignee:alexjbest
0-78359
21 hours ago
0-78359
21 hours ago
26-19830
26 days
33329 mcdoll
author:mcdoll
feat(Analysis): Fourier-based Sobolev spaces We define Sobolev spaces (or Bessel potential spaces). --- - [x] depends on: #33242 - [x] depends on: #32769 - [x] depends on: #33404 - [x] depends on: #33597 - [ ] depends on: #33636 - [x] depends on: #33741 - [x] depends on: #33751 - [ ] depends on: #33752 - [x] depends on: #33776 - [x] depends on: #33859 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-analysis blocked-by-other-PR 936/24 Mathlib/Analysis/Distribution/DerivNotation.lean,Mathlib/Analysis/Distribution/FourierMultiplier.lean,Mathlib/Analysis/Distribution/FourierSchwartz.lean,Mathlib/Analysis/Distribution/Laplacian.lean,Mathlib/Analysis/Distribution/SchwartzSpace.lean,Mathlib/Analysis/Distribution/Sobolev.lean,Mathlib/Analysis/Distribution/TemperedDistribution.lean,Mathlib/Analysis/InnerProductSpace/Laplacian.lean 8 5 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
0-77124
21 hours ago
unknown
unknown
33958 chrisflav
author:chrisflav
feat(AlgebraicGeometry): the small affine étale site From Proetale. --- - [ ] depends on: #33957 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-algebraic-geometry 264/22 Mathlib.lean,Mathlib/AlgebraicGeometry/Sites/AffineEtale.lean,Mathlib/CategoryTheory/Limits/Constructions/Over/Connected.lean,Mathlib/CategoryTheory/Limits/MorphismProperty.lean,Mathlib/CategoryTheory/MorphismProperty/Comma.lean 5 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
0-75424
20 hours ago
unknown
unknown
32745 LTolDe
author:LTolDe
feat(Topology/Algebra): add MulActionConst.lean add Topology/Algebra/MulActionConst.lean introduce class `ContinuousSMulConst` for a scalar multiplication that is continuous in the first argument, in analogy to `ContinuousConstSMul` define `MulAction.ball x U` as the set `U • {x}` given `[SMul G X] (x : X) (U : Set G)` The lemmas shown here will be useful to prove the **Effros Theorem**, see [zulip](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Effros.20Theorem/with/558712441). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author new-contributor t-topology 98/0 Mathlib.lean,Mathlib/Topology/Algebra/MulActionConst.lean 2 6 ['LTolDe', 'github-actions', 'urkud'] dagurtomas
assignee:dagurtomas
0-75342
20 hours ago
2-46172
2 days ago
16-30636
16 days
32692 WilliamCoram
author:WilliamCoram
feat: define multivariate restricted power series We define multivariate restricted power series over a normed ring R, and show the properties that they form a ring when R has the ultrametric property. This work generalises my previous work in #26089 which will need to be refactored. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-ring-theory t-number-theory new-contributor 168/0 Mathlib.lean,Mathlib/RingTheory/MvPowerSeries/Restricted.lean 2 15 ['WilliamCoram', 'erdOne', 'github-actions'] nobody
0-75214
20 hours ago
0-74327
20 hours ago
2-9323
2 days
32807 WilliamCoram
author:WilliamCoram
feat: Define the Gauss norm for MvPowerSeries We adjust the current definition for Gauss norm on power series to work for multivariate power series. If this seems acceptable I can refactor the single variable case. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-ring-theory new-contributor 127/0 Mathlib.lean,Mathlib/RingTheory/MvPowerSeries/GaussNorm.lean 2 11 ['WilliamCoram', 'github-actions', 'mathlib4-merge-conflict-bot', 'vihdzp'] nobody
0-75110
20 hours ago
unknown
unknown
33955 joelriou
author:joelriou
feat(AlgebraicTopology): the fibrant resolution functor up to homotopy This is the dual PR to #33087. --- - [ ] depends on: #33087 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebraic-topology WIP blocked-by-other-PR 443/0 Mathlib.lean,Mathlib/AlgebraicTopology/ModelCategory/CofibrantObjectHomotopy.lean,Mathlib/AlgebraicTopology/ModelCategory/FibrantObjectHomotopy.lean 3 4 ['github-actions', 'joelriou', 'mathlib4-dependent-issues-bot'] nobody
0-73922
20 hours ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-algebra t-category-theory
label:t-algebra$
132/0 Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Ext/DimensionShifting.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/EnoughInjectives.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/EnoughProjectives.lean,Mathlib/Algebra/Homology/ShortComplex/ModuleCat.lean,Mathlib/RingTheory/Noetherian/Basic.lean 6 21 ['Thmoas-Guan', 'erdOne', 'github-actions', 'jcommelin', 'joelriou', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] joelriou
assignee:joelriou
0-73530
20 hours ago
0-73530
20 hours ago
16-14643
16 days
33921 SnirBroshi
author:SnirBroshi
chore(Data/Nat/Factorial): replace `n !` with `(n)!` everywhere Fixes ``Todo: replace occurrences of `n !` with `(n)!` in Mathlib.`` from `Data/Nat/Factorial/Basic.lean`. Only literals are allowed to use factorial unparenthesized, e.g. `5!`. --- The TODO was introduced in #18085, with an accompanying [Zulip discussion](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/precedence.20of.20Nat.2Efactorial) that decided on this. The factorial notation is used in Mathlib on the following kinds of expressions: - `Nat` numerals, e.g. `5`, there are 20 such cases - Identifiers, e.g. `n` or `n.succ` or `l.length` or `p.natDegree`, there are 433 such cases - Structure projection, e.g. `n.1`, there are 20 such cases - Parenthesized expressions, e.g. `(n + k)`, there are 293 such cases - Type ascriptions, e.g. `(n : ℕ)` (these don't count as parenthesized in `Lean.Syntax`), there are [3](https://github.com/leanprover-community/mathlib4/blob/b2f24e70b375e42e5a60251a2f43baa20ca668f1/MathlibTest/norm_num_ext.lean#L625) [such](https://github.com/leanprover-community/mathlib4/blob/b2f24e70b375e42e5a60251a2f43baa20ca668f1/Mathlib/MeasureTheory/Measure/Lebesgue/VolumeOfBalls.lean#L378) [cases](https://github.com/leanprover-community/mathlib4/blob/b2f24e70b375e42e5a60251a2f43baa20ca668f1/Mathlib/MeasureTheory/Measure/Lebesgue/VolumeOfBalls.lean#L384) This PR normalizes everything to use `(...)!` notation, except for numerals which don't require parentheses. Note that structure projections also don't require parentheses but it looks confusing (see [this](https://github.com/leanprover-community/mathlib4/blob/4baa44807be87d9aba67c680ae68c2ba4a7fc29b/Mathlib/Data/Nat/Factorial/NatCast.lean#L106) and [this](https://github.com/leanprover-community/mathlib4/blob/4baa44807be87d9aba67c680ae68c2ba4a7fc29b/Mathlib/NumberTheory/Bernoulli.lean#L150)), so parentheses were added. I used metaprogramming + Python to create this PR; these are the non-formulaic changes: - Deleted the TODO in `Data/Nat/Factorial/Basic.lean` - Fixed 3 comments in `Data/Nat/Factorial/Basic.lean` that used ` !` - The replacement caused these lines to go over the length limit, so I fixed them manually: - `Archive/Imo/Imo2019Q4.lean:84` - `Mathlib/Data/Nat/Choose/Basic.lean:289` - `Mathlib/RingTheory/DividedPowers/RatAlgebra.lean:134` - `Mathlib/RingTheory/Polynomial/ShiftedLegendre.lean:71` In a future PR I'll add a linter that requires parentheses inside factorials for non-numerals, then the whitespace linter will lint against spaces between `)` and `!`. (though the pretty printer's parenthesizer still prefers adding spaces instead of parentheses, not sure how to fix it) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) tech debt t-data 402/401 Archive/Imo/Imo1987Q1.lean,Archive/Imo/Imo2001Q4.lean,Archive/Imo/Imo2019Q4.lean,Mathlib/Algebra/BigOperators/Intervals.lean,Mathlib/Algebra/Group/ForwardDiff.lean,Mathlib/Algebra/Polynomial/Derivative.lean,Mathlib/Algebra/Polynomial/FieldDivision.lean,Mathlib/Algebra/Polynomial/HasseDeriv.lean,Mathlib/Algebra/Polynomial/SumIteratedDerivative.lean,Mathlib/Analysis/Analytic/Binomial.lean,Mathlib/Analysis/Calculus/ContDiff/Bounds.lean,Mathlib/Analysis/Calculus/Deriv/ZPow.lean,Mathlib/Analysis/Calculus/FDeriv/Analytic.lean,Mathlib/Analysis/Calculus/IteratedDeriv/WithinZpow.lean,Mathlib/Analysis/Calculus/Taylor.lean,Mathlib/Analysis/Complex/Exponential.lean,Mathlib/Analysis/Complex/TaylorSeries.lean,Mathlib/Analysis/Distribution/SchwartzSpace.lean,Mathlib/Analysis/Distribution/TemperateGrowth.lean,Mathlib/Analysis/Normed/Algebra/Exponential.lean,Mathlib/Analysis/ODE/PicardLindelof.lean,Mathlib/Analysis/Real/Pi/Irrational.lean,Mathlib/Analysis/Real/Pi/Wallis.lean,Mathlib/Analysis/SpecialFunctions/Exp.lean,Mathlib/Analysis/SpecialFunctions/Gamma/Basic.lean,Mathlib/Analysis/SpecialFunctions/Gamma/Beta.lean,Mathlib/Analysis/SpecialFunctions/Gamma/BohrMollerup.lean,Mathlib/Analysis/SpecialFunctions/OrdinaryHypergeometric.lean,Mathlib/Analysis/SpecialFunctions/Stirling.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Cotangent.lean,Mathlib/Analysis/SpecificLimits/Basic.lean,Mathlib/Analysis/SpecificLimits/Normed.lean,Mathlib/Combinatorics/Enumerative/Bell.lean,Mathlib/Data/Fintype/Perm.lean,Mathlib/Data/List/Permutation.lean,Mathlib/Data/Nat/Choose/Basic.lean,Mathlib/Data/Nat/Choose/Bounds.lean,Mathlib/Data/Nat/Choose/Cast.lean,Mathlib/Data/Nat/Choose/Factorization.lean,Mathlib/Data/Nat/Choose/Multinomial.lean,Mathlib/Data/Nat/Factorial/Basic.lean,Mathlib/Data/Nat/Factorial/BigOperators.lean,Mathlib/Data/Nat/Factorial/DoubleFactorial.lean,Mathlib/Data/Nat/Factorial/NatCast.lean,Mathlib/Data/Nat/Factorial/SuperFactorial.lean,Mathlib/Data/Nat/Multiplicity.lean,Mathlib/Data/Nat/Prime/Factorial.lean,Mathlib/Data/Nat/Prime/Infinite.lean,Mathlib/Data/ZMod/Factorial.lean,Mathlib/GroupTheory/IndexNormal.lean,Mathlib/GroupTheory/Perm/Centralizer.lean,Mathlib/NumberTheory/Bernoulli.lean,Mathlib/NumberTheory/BernoulliPolynomials.lean,Mathlib/NumberTheory/Harmonic/GammaDeriv.lean,Mathlib/NumberTheory/ModularForms/EisensteinSeries/QExpansion.lean,Mathlib/NumberTheory/Padics/PadicVal/Basic.lean,Mathlib/NumberTheory/PrimesCongruentOne.lean,Mathlib/NumberTheory/Transcendental/Lindemann/AnalyticalPart.lean,Mathlib/NumberTheory/Transcendental/Liouville/LiouvilleNumber.lean,Mathlib/NumberTheory/ZetaValues.lean,Mathlib/Probability/Distributions/Poisson.lean,Mathlib/Probability/Moments/MGFAnalytic.lean,Mathlib/RingTheory/DividedPowers/Basic.lean,Mathlib/RingTheory/DividedPowers/Padic.lean,Mathlib/RingTheory/DividedPowers/RatAlgebra.lean,Mathlib/RingTheory/Nilpotent/Exp.lean,Mathlib/RingTheory/Polynomial/HilbertPoly.lean,Mathlib/RingTheory/Polynomial/Pochhammer.lean,Mathlib/RingTheory/Polynomial/ShiftedLegendre.lean,Mathlib/RingTheory/PowerSeries/WellKnown.lean,Mathlib/Tactic/NormNum/NatFactorial.lean,Mathlib/Topology/Algebra/Order/Floor.lean,MathlibTest/GCongr/inequalities.lean,MathlibTest/Simproc/Divisors.lean,MathlibTest/factorial.lean,MathlibTest/norm_num_ext.lean,MathlibTest/positivity.lean 77 1 ['github-actions'] nobody
0-73379
20 hours ago
1-553
1 day ago
1-373
1 day
33960 justus-springer
author:justus-springer
feat(FieldTheory/RatFunc): Generalize lifts/maps to FunLike This was mentioned as a TODO in the file. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra
label:t-algebra$
66/47 Mathlib/FieldTheory/Laurent.lean,Mathlib/FieldTheory/RatFunc/AsPolynomial.lean,Mathlib/FieldTheory/RatFunc/Basic.lean 3 1 ['github-actions'] nobody
0-72740
20 hours ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR t-order merge-conflict 560/477 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 27 ['Vierkantor', 'github-actions', 'linesthatinterlace', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'plp127', 'vihdzp'] YaelDillies
assignee:YaelDillies
0-72326
20 hours ago
94-33826
94 days ago
16-35327
16 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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author new-contributor t-order 255/0 Mathlib.lean,Mathlib/Algebra/BigOperators/Group/Finset/Gaps.lean,Mathlib/Order/Interval/Finset/Gaps.lean 3 6 ['github-actions', 'sgouezel', 'zhuyizheng'] sgouezel
assignee:sgouezel
0-72017
20 hours ago
0-82277
22 hours ago
48-35273
48 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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
214/100 Mathlib/Algebra/Module/LocalizedModule/Basic.lean 1 4 ['erdOne', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant'] nobody
0-71558
19 hours ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra large-import
label:t-algebra$
634/0 Mathlib.lean,Mathlib/GroupTheory/Subgroup/Center.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/NonAbelian.lean,Mathlib/RepresentationTheory/Rep.lean 4 2 ['github-actions', 'mathlib4-merge-conflict-bot'] nobody
0-71110
19 hours ago
0-64366
17 hours ago
0-64186
17 hours
33963 gasparattila
author:gasparattila
feat(Topology/UniformSpace/Closeds): completeness of `(Nonempty)Compacts` This PR generalizes the completeness result of `NonemptyCompacts` from metric spaces to uniform spaces. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology 91/8 Mathlib/Topology/MetricSpace/Closeds.lean,Mathlib/Topology/Sets/Compacts.lean,Mathlib/Topology/UniformSpace/Closeds.lean 3 1 ['github-actions'] nobody
0-71061
19 hours ago
0-68358
18 hours ago
0-68178
18 hours
33044 bryangingechen
author:bryangingechen
ci: also get cache for parent commit cf. https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Mathlib.20has.20moved.20to.20the.20new.20module.20system/near/563452000 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) CI 84/8 .github/build.in.yml,.github/workflows/bors.yml,.github/workflows/build.yml,.github/workflows/build_fork.yml 4 7 ['bryangingechen', 'github-actions', 'jcommelin', 'mathlib-bors'] joneugster
assignee:joneugster
0-70882
19 hours ago
0-70951
19 hours ago
26-31071
26 days
33801 artie2000
author:artie2000
chore: add missing mem lemmas * Add missing `simp` lemmas `mem_foo` where a `simp` lemma `coe_foo` already exists --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta 15/3 Mathlib/AlgebraicGeometry/OpenImmersion.lean,Mathlib/RingTheory/FractionalIdeal/Basic.lean,Mathlib/RingTheory/FractionalIdeal/Extended.lean,Mathlib/Topology/Category/TopCat/Opens.lean,Mathlib/Topology/Sets/Opens.lean 5 7 ['artie2000', 'eric-wieser', 'github-actions'] eric-wieser
assignee:eric-wieser
0-70787
19 hours ago
0-73026
20 hours ago
4-45433
4 days
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-measure-probability 189/0 Mathlib.lean,Mathlib/MeasureTheory/Constructions/UnitInterval.lean,Mathlib/Probability/Kernel/Representation.lean 3 10 ['DavidLedvinka', 'RemyDegenne', 'gaetanserre', 'github-actions', 'mathlib4-merge-conflict-bot'] RemyDegenne
assignee:RemyDegenne
0-70748
19 hours ago
0-69037
19 hours ago
37-63250
37 days
33965 gasparattila
author:gasparattila
feat(Topology/MetricSpace/Closeds): define a metric on `Compacts` This PR defines an `EMetricSpace` instance on `Compacts` using the Hausdorff distance, analogously with the existing metrics on `Closeds` and `NonemptyCompacts`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology 32/0 Mathlib/Topology/MetricSpace/Closeds.lean 1 1 ['github-actions'] nobody
0-69676
19 hours ago
0-64614
17 hours ago
0-64434
17 hours
33854 loefflerd
author:loefflerd
feat(Analysis): generalize normed spaces to normed modules Spin-off from the review process of PR 33723: generalize lots of results about linear/bilinear maps and derivatives to allow more general scalars. --- - [x] depends on: #33723 - [ ] depends on: #33962 WIP blocked-by-other-PR 645/320 Mathlib/Algebra/Module/LinearMap/Defs.lean,Mathlib/Analysis/Analytic/Constructions.lean,Mathlib/Analysis/Analytic/ConvergenceRadius.lean,Mathlib/Analysis/Analytic/Order.lean,Mathlib/Analysis/Calculus/ContDiff/Operations.lean,Mathlib/Analysis/Calculus/Deriv/CompMul.lean,Mathlib/Analysis/Calculus/Deriv/Mul.lean,Mathlib/Analysis/Calculus/DifferentialForm/Basic.lean,Mathlib/Analysis/Calculus/FDeriv/Add.lean,Mathlib/Analysis/Calculus/FDeriv/Equiv.lean,Mathlib/Analysis/Calculus/FDeriv/Mul.lean,Mathlib/Analysis/Calculus/IteratedDeriv/Defs.lean,Mathlib/Analysis/Calculus/IteratedDeriv/Lemmas.lean,Mathlib/Analysis/InnerProductSpace/Calculus.lean,Mathlib/Analysis/Normed/Module/Multilinear/Basic.lean,Mathlib/Analysis/Normed/Operator/Basic.lean,Mathlib/Analysis/Normed/Operator/BoundedLinearMaps.lean,Mathlib/Analysis/Normed/Operator/Mul.lean,Mathlib/Probability/Moments/MGFAnalytic.lean,Mathlib/Topology/Algebra/Module/LinearMap.lean,Mathlib/Topology/Algebra/Module/Multilinear/Basic.lean 21 3 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
0-67943
18 hours ago
unknown
unknown
33712 wangying11123
author:wangying11123
feat(Geometry/Euclidean/Angle/Unoriented/Projection): Add sameray_orthogonalProjection_vsub_of_angle_lt Add sameray_orthogonalProjection_vsub_of_angle_lt `sameray_orthogonalProjection_vsub_of_angle_lt` When an angle is acute, the vector to the orthogonal projection lies in the same ray as the given direction vector. new-contributor t-euclidean-geometry 20/0 Mathlib/Geometry/Euclidean/Angle/Unoriented/Projection.lean 1 2 ['github-actions'] nobody
0-67742
18 hours ago
0-65081
18 hours ago
5-69153
5 days
33907 dupuisf
author:dupuisf
feat(Asymptotics): Show that `f =O[atTop] g` from a recurrence relation This PR introduces two lemmas that are useful to show that `f =O[atTop] g` recursively using a recurrence relation, i.e. by proving that `f n ≤ C * g n` assuming that we know this for smaller values of `n`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis 46/0 Mathlib/Analysis/Asymptotics/Lemmas.lean 1 7 ['ADedecker', 'dupuisf', 'github-actions', 'j-loreaux'] ADedecker
assignee:ADedecker
0-66822
18 hours ago
0-66822
18 hours ago
1-34195
1 day
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-measure-probability merge-conflict 224/136 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 25 ['JonBannon', 'github-actions', 'j-loreaux', 'mathlib4-merge-conflict-bot'] urkud
assignee:urkud
0-66405
18 hours ago
89-59511
89 days ago
12-68529
12 days
33966 gasparattila
author:gasparattila
feat(Topology): characterization of `LocallyConnectedSpace` in terms of `IsTopologicalBasis` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology 13/0 Mathlib/Topology/Connected/LocallyConnected.lean 1 1 ['github-actions'] nobody
0-63850
17 hours ago
0-59912
16 hours ago
0-59732
16 hours
33807 adamtopaz
author:adamtopaz
feat: TypeCat refactor --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-category-theory merge-conflict 114/0 ConstGraph/Main.lean,Mathlib/CategoryTheory/Types/Basic.lean,lakefile.lean 3 2 ['github-actions', 'mathlib4-merge-conflict-bot'] nobody
0-63714
17 hours ago
unknown
unknown
33969 goliath-klein
author:goliath-klein
refactor(PiTensorProduct/{InjectiveNorm, ProjectiveNorm}): Currently, injectiveSeminorm = projectiveSeminorm This is an RFC. Currently, `injectiveSeminorm` is extensionally equal to `projectiveSeminorm`. I'm not sure whether this is by design (it's not documented). # Background Some background, since terminology isn't universal. Based on Chap. 1 of [Diestel et al.](https://www.ams.org/bookstore/pspdf/mbk-52-prev.pdf) On the algebraic tensor product of two Banach spaces X, Y, there are two distinguished norms. First, the "largest reasonable crossnorm": (L1) `‖u‖_∧` = norm of the linear map that sends `b : B(X,Y; 𝕂)` to `(lift b) u`. Here, `B(X,Y; Z)` are the bounded bilinear maps into a normed space `Z`. Equivalently, (L2) `‖u‖_∧ = sup { sum_i ‖x_i‖ ‖y_i‖ | sum_i x_i ⊗ y_i = u }`. Second, there is the "smallest reasonable crossnorm": (S) `‖u‖_∨` = norm of the bilinear map that sends `f : X', g : Y'` to `(f⊗g) u`. The largest / smallest reasonable crossnorms are commonly known as the projective / injective norm. (Though not universally: Grothendieck's "Résumé" and Treves' TVS book use the first, but not the second notion). # Mathlib Mathlib treats `PiTensorProduct`s of seminormed spaces over normed fields. In this context, `projectiveSeminorm` implements (L2). But `injectiveSeminorm u` doesn't implement (S), but the following variant of (L1): (L1') `sup_Z { norm of map sending b : B(X,Y; Z) to (lift b) u }.` In fact, `injectiveSeminorm = projectiveSeminorm `. The upper bound is proven in Mathlib, the lower bound in the PR. The supremum is attained for `Z` the `PiTensorProduct` endowed with the projective seminorm. (Maybe not too surprising, since (L2) = (L1) for Banach spaces, and (L1) is similar to (L1'). The existing `norm_eval_le_injectiveSeminorm` also gets close to this conclusion). # RFC A minimal change would be to add a disclaimer to the docstring of injectiveSeminorm. Here's a suggestion for a larger change. In the current structure, `projectiveSeminorm` is defined first; `injectiveSeminorm` builds on it. Then the theory of an isometric version of `PiTensorProduct.lift` is built on top of `injectiveSeminorm`. One can: * Base all applications on `projectiveSeminorm` instead (using little more than search / replace of "injective" -> "projective"). This seems preferable, because the main results are now established more directly, without the detour via (L1'). * At this point, nothing builds on `injectiveSeminorm` any more. The definition might still be of independent interest. In this case: The optimization over all normed spaces `Z` requires some universe gymnastics (see `norm_eval_le_injectiveSeminorm`). This can be simplified by proving `injectiveSeminorm = projectiveSeminorm` directly. * More radically, `injectiveSeminorm` could be removed. Instead, a proof of (L1) = (L2) assuming [RCLike] could be added. The latter seems more likely to me to have applications. * Formalize (S). The PR implements the first two points and does some initial steps toward the last one. It is meant as an RFC. (The last part in particular isn't ready yet). Comments are very welcome! --- Marked WIP while seeking input from the original author. Co-authored-by: Davood H. H. Tehrani [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-analysis new-contributor 617/457 Mathlib.lean,Mathlib/Analysis/Normed/Module/PiTensorProduct/InjectiveSeminorm.lean,Mathlib/Analysis/Normed/Module/PiTensorProduct/LeastCrossnorm.lean,Mathlib/Analysis/Normed/Module/PiTensorProduct/ProjectiveSeminorm.lean 4 2 ['github-actions', 'goliath-klein'] nobody
0-63274
17 hours ago
unknown
unknown
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`. - [x] Tracing to see what this is doing - [x] Improve the UI of applying the `to_dual_insert_cast` and `to_dual_insert_cast_fun` attributes. - [x] Add tests - [x] Better documentation --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta 512/128 Mathlib.lean,Mathlib/Combinatorics/Quiver/Basic.lean,Mathlib/Order/Basic.lean,Mathlib/Order/Cover.lean,Mathlib/Order/Defs/LinearOrder.lean,Mathlib/Order/Defs/PartialOrder.lean,Mathlib/Order/GaloisConnection/Defs.lean,Mathlib/Order/Interval/Set/Defs.lean,Mathlib/Order/Monotone/Defs.lean,Mathlib/Order/WithBot.lean,Mathlib/Tactic.lean,Mathlib/Tactic/ToDual.lean,Mathlib/Tactic/Translate/Core.lean,Mathlib/Tactic/Translate/ToDual.lean,Mathlib/Tactic/Translate/UnfoldBoundary.lean,MathlibTest/ToDual.lean 16 15 ['JovanGerb', 'fpvandoorn', 'github-actions', 'leanprover-radar', 'mathlib4-merge-conflict-bot', 'vihdzp'] bryangingechen
assignee:bryangingechen
0-63224
17 hours ago
0-58406
16 hours ago
15-9152
15 days
33964 JovanGerb
author:JovanGerb
feat(Order/Interval/Set): `to_dual` for `Iio`/`Iic` This PR tags `Iio`/`Ioi` and `Iic`/`Ici` with `to_dual`. Unfortuately we can't do this yet for `Ioc`/`Ico` and `Ioo` and `Icc`, as we need to have #32438 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 101/219 Mathlib/Order/Interval/Set/Basic.lean,Mathlib/Order/Interval/Set/Defs.lean,Mathlib/Tactic/Translate/ToDual.lean 3 2 ['JovanGerb', 'github-actions'] nobody
0-62993
17 hours ago
unknown
unknown
32355 bjornsolheim
author:bjornsolheim
feat(Geometry/Convex/Cone): define and characterize simplicial pointed cones Define simplicial pointed cones. Prove lemmas about simplicial (and generating simplicial) cones # Notes * I have tried alternative implementations (finite, finset, structure) If one can live with the extensional quantifier the finset seems better. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-convex-geometry new-contributor 116/0 Mathlib.lean,Mathlib/Geometry/Convex/Cone/Pointed.lean,Mathlib/Geometry/Convex/Cone/Simplicial.lean 3 37 ['artie2000', 'bjornsolheim', 'github-actions'] nobody
0-62775
17 hours ago
0-62780
17 hours ago
36-67896
36 days
33936 cameronfreer
author:cameronfreer
feat(NumberTheory/LSeries): add positivity and real-valuedness lemmas for Riemann zeta Add lemmas about the Riemann zeta function for real arguments greater than 1: - `riemannZeta_pos_of_one_lt`: `riemannZeta x` is positive in `ComplexOrder` for real `x > 1` - `riemannZeta_re_pos_of_one_lt`: the real part of `riemannZeta x` is positive for real `x > 1` - `riemannZeta_im_eq_zero_of_one_lt`: `riemannZeta x` has zero imaginary part for real `x > 1` The positivity result follows from `LSeries.positive`, using that the L-series of the constant function 1 equals the Riemann zeta function on the domain of convergence. The key insight is that `0 < z` in `ComplexOrder` simultaneously encodes `z.re > 0` and `z.im = 0` (via `Complex.pos_iff`), so positivity implies real-valuedness. This adds a new import of `Mathlib.NumberTheory.LSeries.Positivity` to `Dirichlet.lean`. The `ComplexOrder` scope is limited to a dedicated nested section to avoid affecting typeclass inference elsewhere. This generalizes `riemannZeta_even_im_eq_zero` from the [Sphere Packing project](https://github.com/thefundamentaltheor3m/Sphere-Packing-Lean/blob/7d4461f1/SpherePacking/ModularForms/Eisenstein.lean#L836-L846), which is now a corollary. new-contributor t-number-theory sphere-packing 25/0 Mathlib/NumberTheory/LSeries/Dirichlet.lean 1 4 ['cameronfreer', 'github-actions', 'metakunt'] nobody
0-62767
17 hours ago
1-27635
1 day ago
1-27455
1 day
33956 joelriou
author:joelriou
feat(AlgebraicTopology/ModelCategory): the right derivability structure We show that the inclusion of the full subcategory of fibrant objects in a model category gives a right derivability structure (with respect to weak equivalences). This PR dualizes #33088 --- - [ ] depends on: #33087 - [ ] depends on: #33088 - [ ] depends on: #33955 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebraic-topology WIP blocked-by-other-PR 786/0 Mathlib.lean,Mathlib/AlgebraicTopology/ModelCategory/CofibrantObjectHomotopy.lean,Mathlib/AlgebraicTopology/ModelCategory/DerivabilityStructureCofibrant.lean,Mathlib/AlgebraicTopology/ModelCategory/DerivabilityStructureFibrant.lean,Mathlib/AlgebraicTopology/ModelCategory/FibrantObjectHomotopy.lean 5 3 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
0-62630
17 hours ago
unknown
unknown
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. The violations found by this linter are fixed in #33068 (merged) and #33148 (merged). Note that the portion of this diff corresponding to the actual linter file is relatively small (+68 -11), and is very similar to the `unusedDecidableInType` linter. The majority of the diff in the linter file itself is factoring out the workaround to lean4#11313 (which is used in both linters); the rest of the diff comes from reorganizing tests and adding tests. --- - [x] depends on: #31142 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) maintainer-merge file-removed 304/46 Mathlib/Tactic/Linter/UnusedInstancesInType.lean,MathlibTest/UnusedInstancesInType/Basic.lean,MathlibTest/UnusedInstancesInType/Decidable.lean,MathlibTest/UnusedInstancesInType/Fintype.lean,MathlibTest/UnusedInstancesInType/FintypeNeedingImport.lean,MathlibTest/UnusedInstancesInType/SetOption.lean 6 15 ['JovanGerb', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'thorimur'] JovanGerb
assignee:JovanGerb
0-62542
17 hours ago
2-48797
2 days ago
40-21713
40 days
28821 yury-harmonic
author:yury-harmonic
refactor(SimpleGraph/Finite): turn `edgeFinset` into a `def` Also add some API lemmas. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics 57/35 Mathlib/Combinatorics/SimpleGraph/Acyclic.lean,Mathlib/Combinatorics/SimpleGraph/Copy.lean,Mathlib/Combinatorics/SimpleGraph/DeleteEdges.lean,Mathlib/Combinatorics/SimpleGraph/Finite.lean,Mathlib/Combinatorics/SimpleGraph/Operations.lean 5 1 ['github-actions'] nobody
0-60920
16 hours ago
unknown
unknown
33962 loefflerd
author:loefflerd
feat(Analysis/Normed): generalize `smul` on cts [multi-]linear maps Allow scalar multiplication by more general types (not just normed fields) that act reasonably on the target of the map. Mostly this just involves swapping typeclass assumptions, but the file `Mathlib/Analysis/Normed/Operator/BoundedLinearMaps.lean` needed a more intensive refactor to separate out the results that are valid over a general base ring from those that really require a `NontriviallyNormedField`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis 212/150 Mathlib/Algebra/Module/LinearMap/Defs.lean,Mathlib/Analysis/Normed/Module/Multilinear/Basic.lean,Mathlib/Analysis/Normed/Operator/Basic.lean,Mathlib/Analysis/Normed/Operator/BoundedLinearMaps.lean,Mathlib/Analysis/Normed/Operator/Mul.lean,Mathlib/Topology/Algebra/Module/LinearMap.lean,Mathlib/Topology/Algebra/Module/Multilinear/Basic.lean 7 3 ['github-actions', 'leanprover-radar', 'loefflerd'] nobody
0-60881
16 hours ago
0-63268
17 hours ago
0-63088
17 hours
33947 urkud
author:urkud
chore: move `Complex.expPartialHomeomorph` Also rename it to `Complex.expOpenPartialHomeomorph`. --- I'm not 100% sure we need to move it. It's a leftover from an older version of #33423. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis 36/26 Mathlib/Analysis/SpecialFunctions/Complex/Log.lean,Mathlib/Analysis/SpecialFunctions/Complex/LogDeriv.lean 2 1 ['github-actions'] nobody
0-60677
16 hours ago
0-57708
15 hours ago
0-57528
15 hours
33971 seewoo5
author:seewoo5
feat(DihedralGroup): center of D_n for odd n \ge 3 trivial --- Center of dihedral group $D_n$ for odd $n \ge 3$ is trivial. Note that initial code was written by Claude Opus 4.5. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-group-theory 22/1 Mathlib/GroupTheory/SpecificGroups/Dihedral.lean 1 1 ['github-actions'] nobody
0-58785
16 hours ago
0-57264
15 hours ago
0-57084
15 hours
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra awaiting-author
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 31 ['github-actions', 'joelriou', 'kckennylau', 'llllvvuu', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] joelriou
assignee:joelriou
0-58008
16 hours ago
57-5544
57 days ago
20-28643
20 days
33919 tb65536
author:tb65536
feat(Algebra/Polynomial/Roots): Action of group on `rootSet` This PR adds an instance for `MulAction G (f.rootSet R)` whenever a `MulSemiringAction G R` satisfies `SMulCommClass G S R`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-ring-theory t-algebra delegated
label:t-algebra$
43/1 Mathlib/Algebra/Polynomial/AlgebraMap.lean,Mathlib/Algebra/Polynomial/Roots.lean 2 11 ['alreadydone', 'eric-wieser', 'github-actions', 'mathlib-bors', 'tb65536'] nobody
0-57480
15 hours ago
0-64607
17 hours ago
0-74129
20 hours
33961 JovanGerb
author:JovanGerb
feat(to_dual): don't translate the order on `Prop` It had been noticed on Zulip that there are lemmas talking about the order on `Prop`, in which `to_dual` should not revert that order. In a sense `Prop` is just as much a fixed type as e.g. `Nat`. This PR adds this check to `shouldTranslate`. I would have expected more translations to break, but it seems that the only thing we need to do is to tell it to not go into the second argument of `Subtype` when checking if a type is fixed. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta 22/13 Mathlib/Tactic/ToAdditive.lean,Mathlib/Tactic/ToDual.lean,Mathlib/Tactic/Translate/Core.lean,MathlibTest/ToDual.lean,MathlibTest/toAdditive.lean 5 1 ['github-actions'] nobody
0-57047
15 hours ago
0-52955
14 hours ago
0-52775
14 hours
33930 chrisflav
author:chrisflav
feat(AlgebraicGeometry): gluing colimits in `P.Over ⊤ S` Let `D : J ⥤ P.Over ⊤ S` be a diagram and `𝒰` a locally directed open cover of `S` (e.g., the cover of all affine opens of `S`). Suppose the restrictions of `D` to `Dᵢ : J ⥤ P.Over ⊤ (𝒰.X i)` have a colimit for every `i`, then we show that also `D` has a colimit under suitable assumptions. This can be used to reduce existence of certain colimits in `P.Over ⊤ S` to the case where `S` is affine. From Pi1. --- - [ ] depends on: #33898 - [ ] depends on: #33932 - [ ] depends on: #33931 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebraic-geometry 578/11 Mathlib.lean,Mathlib/AlgebraicGeometry/ColimitsOver.lean,Mathlib/AlgebraicGeometry/Cover/Directed.lean,Mathlib/AlgebraicGeometry/Gluing.lean,Mathlib/AlgebraicGeometry/RelativeGluing.lean,Mathlib/CategoryTheory/MorphismProperty/Composition.lean,Mathlib/CategoryTheory/MorphismProperty/OverAdjunction.lean 7 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
0-56273
15 hours ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-computability new-contributor awaiting-author awaiting-CI 405/7 Mathlib/Computability/NFA.lean 1 16 ['YaelDillies', 'ctchou', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] YaelDillies
assignee:YaelDillies
0-54103
15 hours ago
0-54103
14 hours ago
43-73349
43 days
33928 jsm28
author:jsm28
feat(Combinatorics/Tiling/TileSet): indexed families of tiles Define the type `TileSet` for indexed families of tiles (in a discrete context), and some associated definitions (including `symmetryGroup`) and API lemmas. `TileSet` can be used for tilings of the whole space; for tilings of part of the space; for patches of tiles (extracted from a tiling by considering tiles meeting some set of points, or considered on their own without extracting from a tiling); for multiple tilings (covering the space more than once). In particular, the fact that people study multiple tilings provides a clear justification for using indexed families rather than sets of tiles, and basic definitions and API lemmas generally work for all these different uses of `TileSet` (sometimes with weak constraints such as tiles being finite, nonempty and only having finitely many tiles meeting any point of the space). Definitions for saying e.g. "this `TileSet` is a tiling of the whole space" are to be included in subsequent files in subsequent PRs. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics 476/0 Mathlib.lean,Mathlib/Combinatorics/Tiling/TileSet.lean 2 4 ['github-actions', 'jsm28', 'vihdzp'] nobody
0-53892
14 hours ago
1-37575
1 day ago
1-37395
1 day
33744 bilichboris
author:bilichboris
feat(RingTheory): Class Group of a Unique Factorization Domain is trivial Add a theorem that the class group of a unique factorization domain is trivial. Together with the PR relating `ClassGroup` to `PicardGroup`, this will close a TODO in `Mathlib.RingTheory.PicardGroup` that the Picard Group of a UFD is trivial. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-ring-theory new-contributor 350/1 Mathlib.lean,Mathlib/RingTheory/FractionalIdeal/Operations.lean,Mathlib/RingTheory/PicardGroup.lean,Mathlib/RingTheory/UniqueFactorizationDomain/ClassGroup.lean 4 14 ['alreadydone', 'bilichboris', 'github-actions', 'jcommelin', 'kim-em', 'tb65536'] erdOne
assignee:erdOne
0-53563
14 hours ago
1-1376
1 day ago
5-76142
5 days
33397 themathqueen
author:themathqueen
feat(Topology/Algebra/Star/LinearMap): intrinsic star for continuous linear maps --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-topology
label:t-algebra$
104/0 Mathlib.lean,Mathlib/Topology/Algebra/Star/LinearMap.lean 2 11 ['github-actions', 'j-loreaux', 'themathqueen'] ocfnash
assignee:ocfnash
0-50065
13 hours ago
0-84550
23 hours ago
15-62782
15 days
29942 smmercuri
author:smmercuri
feat(InfinitePlace/Completion): embeddings of `w.Completion` factor through embeddings of `v.Completion` when `w` extends `v` If `w : InfinitePlace L` and `v : InfinitePlace K` to `L` are such that we have `Algebra v.Completion w.Completion`, then `extensionEmbedding w : L →+* ℂ` factors through `extensionEmbedding v : K →+* ℂ` (provided the algebras are well behaved). --- - [x] depends on: #27978 - [x] depends on: #29969 - [x] depends on: #29944 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) FLT 102/15 Mathlib/Analysis/Normed/Field/WithAbs.lean,Mathlib/NumberTheory/NumberField/InfinitePlace/Completion.lean,Mathlib/NumberTheory/NumberField/InfinitePlace/Embeddings.lean,Mathlib/Topology/MetricSpace/Completion.lean 4 6 ['github-actions', 'joelriou', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
0-49364
13 hours ago
0-48456
13 hours ago
47-37031
47 days
25899 pfaffelh
author:pfaffelh
feat(Topology/Compactness/CompactSystem): introduce compact Systems A compact system is a set systems with the property that, whenever a countable intersections of sets in the set system is empty, there is a finite subset of sets with empty intersection. These are needed e.g. in measure theory if one wants to show sigma-additivity of a set function on a ring. * Main result: The set of sets which are either compact and closed, or `univ`, is a compact system. * Introduce `Dissipate s x := ⋂ y ≤ x, s y` (Data/Set/Dissipate), which is parallel to Data/Set/Accumulate. Co-authored-by: Rémy Degenne remydegenne@gmail.com --- *This PR continues the work from #24541.* *Original PR: https://github.com/leanprover-community/mathlib4/pull/24541* merge-conflict awaiting-author t-topology brownian 387249/162147 .docker/gitpod-blueprint/Dockerfile,.docker/gitpod/Dockerfile,.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/check_pr_titles.yaml,.github/workflows/commit_verification.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/Hairer.lean,Archive/Imo/Imo1959Q2.lean,Archive/Imo/Imo1960Q1.lean,Archive/Imo/Imo1960Q2.lean,Archive/Imo/Imo1961Q3.lean,Archive/Imo/Imo1962Q1.lean,Archive/Imo/Imo1962Q4.lean,Archive/Imo/Imo1972Q5.lean,Archive/Imo/Imo1975Q1.lean,Archive/Imo/Imo1982Q1.lean,Archive/Imo/Imo1982Q3.lean,Archive/Imo/Imo1985Q2.lean,Archive/Imo/Imo1987Q1.lean,Archive/Imo/Imo1988Q6.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/Imo2001Q6.lean,Archive/Imo/Imo2005Q3.lean,Archive/Imo/Imo2005Q4.lean,Archive/Imo/Imo2006Q3.lean,Archive/Imo/Imo2008Q2.lean,Archive/Imo/Imo2008Q3.lean,Archive/Imo/Imo2008Q4.lean,Archive/Imo/Imo2010Q5.lean,Archive/Imo/Imo2011Q3.lean,Archive/Imo/Imo2013Q1.lean,Archive/Imo/Imo2013Q5.lean,Archive/Imo/Imo2015Q6.lean,Archive/Imo/Imo2019Q2.lean,Archive/Imo/Imo2019Q4.lean,Archive/Imo/Imo2021Q1.lean,Archive/Imo/Imo2024Q1.lean,Archive/Imo/Imo2024Q2.lean,Archive/Imo/Imo2024Q3.lean,Archive/Imo/Imo2024Q5.lean,Archive/Imo/Imo2024Q6.lean,Archive/Imo/Imo2025Q3.lean,Archive/Imo/README.md,Archive/Kuratowski.lean,Archive/MiuLanguage/Basic.lean,Archive/OxfordInvariants/Summer2021/Week3P1.lean,Archive/Sensitivity.lean 7913 38 ['github-actions', 'mathlib4-merge-conflict-bot', 'pfaffelh', 'sgouezel'] PatrickMassot
assignee:PatrickMassot
0-47591
13 hours ago
117-79689
117 days ago
70-63338
70 days
33282 AntoineChambert-Loir
author:AntoineChambert-Loir
feat(LinearAlgebra/Center): description of the center of the algebra of endomorphisms Describe the center of the algebra of endomorphisms: under suitable assumptions (eg, over a field), they correspond to - endomorphisms that commute with elementary transvections - endomorphisms `f` such that `v` and `f v` are linearly dependent, for all `v`. If `V` is an `R`-module, we say that an endomorphism `f : Module.End R V` is a *homothety* with central ratio if there exists `a ∈ Set.center R` such that `f x = a • x` for all `x`. By docs#Module.End.mem_subsemiringCenter_iff, these linear maps constitute the center of `Module.End R V`. (When `R` is commutative, we can write `f = a • LinearMap.id`.) In what follows, `V` is assumed to be a free `R`-module. * `LinearMap.commute_transvections_iff_of_basis`: if an endomorphism `f : V →ₗ[R] V` commutes with every elementary transvections (in a given basis), then it is an homothety whose central ratio. (Assumes that the basis is provided and has a non trivial set of indices.) * `LinearMap.exists_eq_smul_id_of_forall_notLinearIndependent`: over a commutative ring `R` which is a domain, an endomorphism `f : V →ₗ[R] V` of a free domain such that `v` and `f v` are not linearly independent, for all `v : V`, is a homothety. * `LinearMap.exists_mem_center_apply_eq_smul_of_forall_notLinearIndependent`: a variant that does not assume that `R` is commutative. Then the homothety has central ratio. * `LinearMap.exists_mem_center_apply_eq_smul_of_forall_notLinearIndependent_of_basis`: a variant that does not assume that `R` has the strong rank condition, but requires a basis. Note. In the noncommutative case, the last two results do not hold when the rank is equal to 1. Indeed, right multiplications with noncentral ratio of the `R`-module `R` satisfy the property that `f v` and `v` are linearly independent, for all `v : V`, but they are not left multiplication by some element. --- - [x] depends on: #33101 - [x] depends on: #33301 (for the mention of docs#Module.End.mem_subsemiringCenter_iff) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
263/4 Mathlib.lean,Mathlib/Algebra/Ring/Subring/Basic.lean,Mathlib/Algebra/Ring/Subsemiring/Basic.lean,Mathlib/GroupTheory/Submonoid/Center.lean,Mathlib/LinearAlgebra/Center.lean,Mathlib/LinearAlgebra/QuadraticForm/Basic.lean 6 20 ['AntoineChambert-Loir', 'eric-wieser', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'themathqueen'] dagurtomas
assignee:dagurtomas
0-47056
13 hours ago
0-44512
12 hours ago
6-82340
6 days
33259 YuvalFilmus
author:YuvalFilmus
feat(Trigonometric/Chebyshev/Extremal): Chebyshev polynomials are extremal in terms of leading coefficient We prove that among all degree n polynomials P such that |P(x)|≤1 for all |x|≤1, the n'th Chebyshev polynomial uniquely maximized the leading coefficient. A subsequent PR will prove a similar property for iterated derivatives evaluated at points x≥1. --- - [ ] depends on: #33194 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis blocked-by-other-PR 255/20 Mathlib.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Chebyshev/Extremal.lean,Mathlib/LinearAlgebra/Lagrange.lean 3 22 ['YuvalFilmus', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'sgouezel'] sgouezel
assignee:sgouezel
0-45237
12 hours ago
7-48212
7 days ago
12-68666
12 days
33914 Vierkantor
author:Vierkantor
fix(Tactic/Linter): support Verso docstrings in header style linter This PR teaches the header style linter to also allow a Verso docstring for the first module docstring. On a file with the option `doc.verso` set to `true` (set this in the Lakefile), the header style linter previously thought there were no docstrings at all, and complained about a missing module docstring. Also fix a docstring that Verso failed to parse (a bit of text should have been code). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-linter delegated 58/5 Mathlib/Tactic/Linter/Header.lean,MathlibTest/HeaderFail.lean,MathlibTest/VersoHeader.lean 3 9 ['Vierkantor', 'adomani', 'github-actions', 'grunweg', 'mathlib-bors'] nobody
0-44868
12 hours ago
unknown
unknown
33833 JovanGerb
author:JovanGerb
feat(reassoc): tag the generated declaration with `to_dual none` This PR adds the feature to `@[reassoc]` that it tags the generated declaration with `to_dual none` whenever the original declaration has been tagged with `to_dual`. In practice, this means that when mixing uses of `to_dual` and `reassoc`, the `to_dual` should come before the `reassoc`, or as `to_dual (attr := reassoc)`. In the rare case that the original expression is not tagged with `to_dual` because it is entirely self dual, we will need to manually tag the generated lemma with `to_dual none`. To do this, `addRelatedDecl` is refactored so that the translated name needs to be supplied, instead of just a pre and postfix. This extra flexibility may come in handy later. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta 35/14 Mathlib/Tactic/CategoryTheory/Elementwise.lean,Mathlib/Tactic/CategoryTheory/Reassoc.lean,Mathlib/Tactic/CategoryTheory/ToApp.lean,Mathlib/Tactic/ToFun.lean,Mathlib/Tactic/Translate/ToDual.lean,Mathlib/Util/AddRelatedDecl.lean,MathlibTest/CategoryTheory/Reassoc.lean 7 2 ['JovanGerb', 'github-actions'] nobody
0-44632
12 hours ago
0-41822
11 hours ago
4-16573
4 days
33683 joelriou
author:joelriou
feat(AlgebraicTopology/SimplicialSet): the simplicial homotopy induced by an homotopy In this PR, we show that a homotopy between morphisms of simplicial sets (given as a morphism `X ⊗ Δ[1] ⟶ Y`) induces a "combinatorial" simplicial homotopy. WIP --- - [ ] depends on: #32881 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR t-algebraic-topology WIP 733/0 Mathlib.lean,Mathlib/AlgebraicTopology/SimplicialObject/SimplicialHomotopy.lean,Mathlib/AlgebraicTopology/SimplicialSet/Monoidal.lean,Mathlib/AlgebraicTopology/SimplicialSet/ProdStdSimplex.lean,Mathlib/AlgebraicTopology/SimplicialSet/ProdStdSimplexOne.lean,Mathlib/AlgebraicTopology/SimplicialSet/SimplicialHomotopy.lean,Mathlib/AlgebraicTopology/SimplicialSet/StdSimplex.lean,Mathlib/AlgebraicTopology/SimplicialSet/StdSimplexOne.lean 8 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
0-43519
12 hours ago
unknown
unknown
33834 JovanGerb
author:JovanGerb
feat(CategoryTheory/NatTrans): use to_dual This PR tags `NatTrans` with `to_dual`. The two functor arguments get swapped because the underlying `NatTrans.app` has its direction swapped. Translating the `naturality` field is slightly awkward. We need to define a constant `naturality'` (analogously to `Category.assoc') --- - [ ] depends on: #33237 - [ ] depends on: #33777 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 11/3 Mathlib/CategoryTheory/NatTrans.lean 1 3 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
0-43044
11 hours ago
0-40651
11 hours ago
0-40471
11 hours
33974 mckoen
author:mckoen
feat(CategoryTheory/Functor): pushout-products and pullback-powers Adds basic API for pushout-products and pullback-powers (also called the Leibniz constructions). Moves the API for `PushoutObjObj` and `PullbackObjObj` from `Mathlib.CategoryTheory.LiftingProperties.ParametrizedAdjunction` and uses this API to define the Leibniz bifunctors on the associated arrow categories. - https://ncatlab.org/nlab/show/pushout-product - https://ncatlab.org/nlab/show/pushout-product --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-category-theory 466/122 Mathlib.lean,Mathlib/CategoryTheory/LiftingProperties/ParametrizedAdjunction.lean,Mathlib/CategoryTheory/Limits/Shapes/Pullback/PullbackObjObj.lean 3 1 ['github-actions'] nobody
0-42518
11 hours ago
unknown
unknown
25273 YaelDillies
author:YaelDillies
refactor: make `MonoidAlgebra` into a one-field structure --- - [x] depends on: #26732 - [x] depends on: #28407 - [x] depends on: #28460 - [x] depends on: #28511 - [x] depends on: #29207 - [x] depends on: #30877 - [x] depends on: #31143 - [x] depends on: #31144 - [x] depends on: #32253 - [x] depends on: #32254 - [x] depends on: #32398 - [x] depends on: #32501 - [x] depends on: #32508 - [x] depends on: #32562 - [x] depends on: #32588 - [x] depends on: #32591 - [x] depends on: #32592 - [x] depends on: #32604 - [x] depends on: #32965 - [x] depends on: #33093 - [x] depends on: #33094 - [x] depends on: #33099 - [x] depends on: #33137 - [x] depends on: #33139 - [x] depends on: #33141 - [x] depends on: #33452 - [x] depends on: #33453 - [x] depends on: #33482 - [x] depends on: #33492 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-algebra large-import
label:t-algebra$
1460/1372 Mathlib/Algebra/FreeAlgebra/Cardinality.lean,Mathlib/Algebra/MonoidAlgebra/Basic.lean,Mathlib/Algebra/MonoidAlgebra/Cardinal.lean,Mathlib/Algebra/MonoidAlgebra/Defs.lean,Mathlib/Algebra/MonoidAlgebra/Degree.lean,Mathlib/Algebra/MonoidAlgebra/Division.lean,Mathlib/Algebra/MonoidAlgebra/Grading.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/Algebra/MonoidAlgebra/ToDirectSum.lean,Mathlib/Algebra/MvPolynomial/Basic.lean,Mathlib/Algebra/MvPolynomial/Cardinal.lean,Mathlib/Algebra/MvPolynomial/CommRing.lean,Mathlib/Algebra/MvPolynomial/Degrees.lean,Mathlib/Algebra/MvPolynomial/Derivation.lean,Mathlib/Algebra/MvPolynomial/Division.lean,Mathlib/Algebra/MvPolynomial/Equiv.lean,Mathlib/Algebra/MvPolynomial/Eval.lean,Mathlib/Algebra/MvPolynomial/Rename.lean,Mathlib/Algebra/Polynomial/Basic.lean,Mathlib/Algebra/Polynomial/Basis.lean,Mathlib/Algebra/Polynomial/Cardinal.lean,Mathlib/Algebra/Polynomial/Coeff.lean,Mathlib/Algebra/Polynomial/Degree/Definitions.lean,Mathlib/Algebra/Polynomial/Eval/Coeff.lean,Mathlib/Algebra/Polynomial/Laurent.lean,Mathlib/Algebra/Polynomial/Module/Basic.lean,Mathlib/Algebra/Polynomial/OfFn.lean,Mathlib/Algebra/Polynomial/Reverse.lean,Mathlib/Algebra/Polynomial/UnitTrinomial.lean,Mathlib/Algebra/Ring/Subring/IntPolynomial.lean,Mathlib/Analysis/Fourier/BoundedContinuousFunctionChar.lean,Mathlib/LinearAlgebra/Finsupp/VectorSpace.lean,Mathlib/LinearAlgebra/FreeAlgebra.lean,Mathlib/RepresentationTheory/Basic.lean,Mathlib/RepresentationTheory/Rep.lean,Mathlib/RingTheory/Coalgebra/MonoidAlgebra.lean,Mathlib/RingTheory/Extension/Generators.lean,Mathlib/RingTheory/FiniteType.lean,Mathlib/RingTheory/Finiteness/Finsupp.lean,Mathlib/RingTheory/HopfAlgebra/MonoidAlgebra.lean,Mathlib/RingTheory/MvPolynomial/Basic.lean,Mathlib/RingTheory/MvPolynomial/EulerIdentity.lean,Mathlib/RingTheory/MvPolynomial/FreeCommRing.lean,Mathlib/RingTheory/MvPolynomial/Homogeneous.lean,Mathlib/RingTheory/MvPolynomial/IrreducibleQuadratic.lean,Mathlib/RingTheory/MvPolynomial/Symmetric/Defs.lean,Mathlib/RingTheory/MvPolynomial/WeightedHomogeneous.lean,Mathlib/RingTheory/Polynomial/Basic.lean,Mathlib/RingTheory/Polynomial/Opposites.lean,Mathlib/RingTheory/TensorProduct/MvPolynomial.lean 56 78 ['JovanGerb', 'YaelDillies', 'alreadydone', 'eric-wieser', 'fpvandoorn', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
0-42202
11 hours ago
unknown
unknown
33846 ocfnash
author:ocfnash
feat: the rank of the ℤ-span of the roots of a root system is the dimension Essentially all the work goes into proving the key lemma `Submodule.finrank_span_eq_finrank_span`. This needs assumptions that the relevant algebra `A` is flat as an `R`-module and also that the algebra map `R → A` is a ring epimorphism in the categorical sense (and that `R` is a principal ideal domain). In the actual application `R = ℤ` and `A = ℚ`, and a much shorter direct proof is possible but this seemed like a good time to develop the general theory a bit more. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra large-import
label:t-algebra$
323/33 Mathlib.lean,Mathlib/Algebra/Algebra/Epi.lean,Mathlib/Algebra/Category/Ring/Epi.lean,Mathlib/LinearAlgebra/RootSystem/IsValuedIn.lean,Mathlib/LinearAlgebra/Span/TensorProduct.lean,Mathlib/RingTheory/TensorProduct/Finite.lean,Mathlib/Tactic/Linter/DirectoryDependency.lean 7 6 ['github-actions', 'jcommelin', 'ocfnash'] nobody
0-41403
11 hours ago
0-41833
11 hours ago
1-10684
1 day
33979 adomani
author:adomani
ci: add `splice-bot` action Adds a CI action that inspects review comments. If a review comment selects at least one line and contains the string `splice-bot` at the start of some line, then the bot will create a PR with just the changes to the selected file, clearing all history. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) CI 16/0 .github/workflows/splice_bot.yaml 1 2 ['bryangingechen', 'github-actions'] bryangingechen
assignee:bryangingechen
0-41314
11 hours ago
unknown
unknown
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: ![](https://ncatlab.org/nlab/files/frobenius_laws.jpg) 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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-ring-theory awaiting-author blocked-by-other-PR 163/0 Mathlib.lean,Mathlib/RingTheory/Coalgebra/Frobenius.lean 2 19 ['YaelDillies', 'erdOne', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'themathqueen'] alreadydone
assignee:alreadydone
0-41174
11 hours ago
46-59940
46 days ago
30-18358
30 days
33916 AntoineChambert-Loir
author:AntoineChambert-Loir
feat(LinearAlgebra/SpecialLinearGroup/Simple): simplicity of the projective special linear group. Let `K` be a field and `V` be a `K`-vector space. * `SpecialLinearGroup.isQuasiSimpleGroup`: if `finrank K V` is at least 3, or if `finrank K V = 2` and `K` has at least 4 elements, then `SpecialLinearGroup K V` is quasi-simple, namely, the quotient group `SpecialLinearGroup K V ⧸ Subgroup.center (SpecialLinearGroup K V)` is simple. --- - [ ] depends on: #33347 - [ ] depends on: #33348 - [ ] depends on: #33387 - [ ] depends on: #33282 - [ ] depends on: #33392 - [ ] depends on: #33402 - [ ] depends on: #33485 - [ ] depends on: #32757 - [ ] depends on: #33560 - [ ] depends on: #33692 - [ ] depends on: #33882 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) file-removed large-import blocked-by-other-PR 3527/239 Mathlib.lean,Mathlib/GroupTheory/Commutator/Basic.lean,Mathlib/LinearAlgebra/Basis/Fin.lean,Mathlib/LinearAlgebra/Center.lean,Mathlib/LinearAlgebra/Determinant.lean,Mathlib/LinearAlgebra/Dual/Defs.lean,Mathlib/LinearAlgebra/FiniteDimensional/Basic.lean,Mathlib/LinearAlgebra/FiniteDimensional/Lemmas.lean,Mathlib/LinearAlgebra/LinearIndependent/Lemmas.lean,Mathlib/LinearAlgebra/Projectivization/Action.lean,Mathlib/LinearAlgebra/Projectivization/Basic.lean,Mathlib/LinearAlgebra/SpecialLinearGroup.lean,Mathlib/LinearAlgebra/SpecialLinearGroup/Simple.lean,Mathlib/LinearAlgebra/Transvection.lean,Mathlib/LinearAlgebra/Transvection/Basic.lean,Mathlib/LinearAlgebra/Transvection/Generation.lean,Mathlib/LinearAlgebra/Transvection/SpecialLinearGroup.lean 17 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
0-40999
11 hours ago
unknown
unknown
33129 Paul-Lez
author:Paul-Lez
feat(Tactic/Simproc/VecPerm): Add simproc for permuting entries of a vector --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta 131/0 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Simproc/VecPerm.lean,MathlibTest/Simproc/VecPerm.lean 4 16 ['JovanGerb', 'Paul-Lez', 'github-actions', 'ocfnash'] thorimur
assignee:thorimur
0-40244
11 hours ago
2-37684
2 days ago
23-22246
23 days
33221 stepan2698-cpu
author:stepan2698-cpu
feat: definition of an intertwining map Adds the definition of an intertwining map of representations, with an instance of an A-module structure. Proves that a multiplication by a central element is an intertwining map. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra new-contributor
label:t-algebra$
162/11 Mathlib.lean,Mathlib/RepresentationTheory/Intertwining.lean,Mathlib/RepresentationTheory/Subrepresentation.lean 3 6 ['github-actions', 'ocfnash'] ocfnash
assignee:ocfnash
0-40193
11 hours ago
5-58118
5 days ago
12-31186
12 days
33466 Shreyas4991
author:Shreyas4991
refactor(Combinatorics/Digraph): add vertex sets --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics 443/53 Mathlib/Combinatorics/Digraph/Basic.lean,Mathlib/Combinatorics/Digraph/Orientation.lean 2 57 ['Shreyas4991', 'SnirBroshi', 'copilot-pull-request-reviewer', 'github-actions', 'mathlib4-merge-conflict-bot', 'vihdzp'] nobody
0-39853
11 hours ago
0-63676
17 hours ago
1-73621
1 day
33953 vihdzp
author:vihdzp
feat: IncompRel.ne Used in the CGT repo. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order easy 6/3 Mathlib/Order/Comparable.lean 1 5 ['eric-wieser', 'github-actions', 'vihdzp'] nobody
0-39751
11 hours ago
0-36709
10 hours ago
0-85725
23 hours
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. From https://github.com/urkud/SardMoreira --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-measure-probability 207/0 Mathlib.lean,Mathlib/MeasureTheory/Integral/IntervalIntegral/DistLEIntegral.lean 2 1 ['github-actions'] nobody
0-39366
10 hours ago
5-11074
5 days ago
48-46011
48 days
33950 vihdzp
author:vihdzp
feat(Order/UpperLower/Basic): use `to_dual` - part 1 --- The rest of these tags are contingent on #33760 and #32438. - [ ] depends on: #33961 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR t-order 27/92 Mathlib/Order/UpperLower/Basic.lean 1 4 ['JovanGerb', 'github-actions', 'mathlib4-dependent-issues-bot'] nobody
0-39130
10 hours ago
0-39131
10 hours ago
0-53122
14 hours
33402 AntoineChambert-Loir
author:AntoineChambert-Loir
feat(LinearAlgebra/Transvection/Generation): prove exceptional case in Dieudonné's theorem Establish the fourth part of Dieudonné's theorem: is a linear equivalence is exceptional, it is the product of `finrank K (V ⧸ e.fixedSubmodule)` transvections and one dilatransvection. --- - [ ] depends on: #33348 - [ ] depends on: #33347 - [ ] depends on: #33387 - [ ] depends on: #33282 - [ ] depends on: #33392 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) file-removed t-algebra blocked-by-other-PR
label:t-algebra$
1569/222 Mathlib.lean,Mathlib/LinearAlgebra/Center.lean,Mathlib/LinearAlgebra/Determinant.lean,Mathlib/LinearAlgebra/FiniteDimensional/Lemmas.lean,Mathlib/LinearAlgebra/LinearIndependent/Lemmas.lean,Mathlib/LinearAlgebra/Transvection.lean,Mathlib/LinearAlgebra/Transvection/Basic.lean,Mathlib/LinearAlgebra/Transvection/Generation.lean 8 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
0-39039
10 hours ago
unknown
unknown
33485 AntoineChambert-Loir
author:AntoineChambert-Loir
feat(LinearAlgebra/Transvection/Generation): prove the third part of Dieudonné's theorem Prove the third part of Dieudonné's theorem : if `e : V ≃ₗ[K] V` is a product of `finrank K (V ⧸ e.fixedSubmodule) - 1` transvections and one dilatransvection, then it is not exceptional. Actually, we prove something slightly stronger : if `e : V ≃ₗ[K] V` is a product of a transvection and of `finrank K (V ⧸ e.fixedSubmodule) - 1` dilatransvections, then it is not exceptional. --- - [ ] depends on: #33347 - [ ] depends on: #33348 - [ ] depends on: #33387 - [ ] depends on: #33282 - [ ] depends on: #33392 - [ ] depends on: #33402 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) file-removed t-algebra blocked-by-other-PR
label:t-algebra$
2016/222 Mathlib.lean,Mathlib/LinearAlgebra/Center.lean,Mathlib/LinearAlgebra/Determinant.lean,Mathlib/LinearAlgebra/FiniteDimensional/Lemmas.lean,Mathlib/LinearAlgebra/LinearIndependent/Lemmas.lean,Mathlib/LinearAlgebra/Transvection.lean,Mathlib/LinearAlgebra/Transvection/Basic.lean,Mathlib/LinearAlgebra/Transvection/Generation.lean 8 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
0-38996
10 hours ago
unknown
unknown
33560 AntoineChambert-Loir
author:AntoineChambert-Loir
feat(LinearAlgebra/Transvection/Generation): a linear equivalence is the product of dilatransvections Prove that a linear equivalence `e` is the product of `V ⧸ e.fixedSubmodule` dilatransvections. (It cannot be a product of less.) --- - [ ] depends on: #33347 - [ ] depends on: #33348 - [ ] depends on: #33387 - [ ] depends on: #33282 - [ ] depends on: #33392 - [ ] depends on: #33402 - [ ] depends on: #33485 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) file-removed t-algebra blocked-by-other-PR
label:t-algebra$
2129/222 Mathlib.lean,Mathlib/LinearAlgebra/Center.lean,Mathlib/LinearAlgebra/Determinant.lean,Mathlib/LinearAlgebra/FiniteDimensional/Lemmas.lean,Mathlib/LinearAlgebra/LinearIndependent/Lemmas.lean,Mathlib/LinearAlgebra/Transvection.lean,Mathlib/LinearAlgebra/Transvection/Basic.lean,Mathlib/LinearAlgebra/Transvection/Generation.lean 8 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
0-38959
10 hours ago
unknown
unknown
33923 grunweg
author:grunweg
fix: example of GL(V) being a Lie group The doc-string was missing a smoothness parameter. Fix this, and copy-paste this example into the file to ensure it does not regress in the future. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-differential-geometry easy 5/3 Mathlib/Geometry/Manifold/Instances/UnitsOfNormedAlgebra.lean 1 9 ['github-actions', 'grunweg', 'ocfnash'] nobody
0-38883
10 hours ago
0-36487
10 hours ago
1-48108
1 day
33693 yoh-tanimoto
author:yoh-tanimoto
feat(Mathlib/Analysis/Normed/Module): add instances of `CompleteSpace` for `Submodules` and `ClosedSubmodule` add an instance of `CompleteSpace` for a `Submodule` of a Banach space `[NormedField 𝕜] [NormedAddCommGroup E] [NormedSpace 𝕜 E] [CompleteSpace E]` which `IsClosed`. ~~In this relation, convert a lemma showing `IsClosed` to an instance for `ClosedSubmodule`.~~ motivation: Together with #28709, this makes it automatic that a `ClosedSubmodule` in a Hilbert space `HasOrthogonalProjection`. discussion: https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/.60CompleteSpace.60.20for.20closed.20subtypes.20in.20a.20.60CompleteSpace.60 19/1 Mathlib/Analysis/InnerProductSpace/Orthogonal.lean,Mathlib/Topology/Algebra/Module/Basic.lean,Mathlib/Topology/Algebra/Module/ClosedSubmodule.lean 3 8 ['github-actions', 'leanprover-radar', 'sgouezel', 'yoh-tanimoto'] jcommelin
assignee:jcommelin
0-38547
10 hours ago
0-45052
12 hours ago
7-17198
7 days
33980 martinwintermath
author:martinwintermath
feat(RingTheory/Finiteness/Basic): add lemmas for restricting scalars This PR adds three lemmas that transfer `Submodule.FG` across restricting scalars from a semiring `A` to a semiring `R` under the assumption `Module.Finite R A` . This includes * `fg_restrictScalars` which proves that `restrictScalars` preserves `FG` * `fg_restrictScalars_iff` as the iff version of the above * `span_submodule_fg_of_fg` which proves that the `A`-span of an `FG` `R`-submodule is `FG`. The PR also contains the following changes to related lemmas: * renaming `fg_restrictScalars` to `fg_restrictScalars_of_surjective` emphasizing the hypothesis `Function.Surjective (algebraMap R A)` * adding a `sections RestrictScalars` that also contains the above lemma * restructuring variables in the above section --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-ring-theory new-contributor 39/9 Mathlib/RingTheory/Finiteness/Basic.lean,Mathlib/RingTheory/Finiteness/Ideal.lean 2 1 ['github-actions'] nobody
0-37844
10 hours ago
0-34171
9 hours ago
0-33991
9 hours
33194 YuvalFilmus
author:YuvalFilmus
feat(LinearAlgebra/Lagrange): refactored proof of leadingCoeff_eq_sum The proof of `leadingCoeff_eq_sum` was slightly refactored. A subsequent PR will use the refactored parts to prove a formula for the iterated derivative of a polynomial at a point. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
15/17 Mathlib/LinearAlgebra/Lagrange.lean 1 11 ['Ruben-VandeVelde', 'YuvalFilmus', 'github-actions', 'sgouezel', 'vlad902'] dagurtomas
assignee:dagurtomas
0-37683
10 hours ago
0-31612
8 hours ago
23-59763
23 days
33236 JovanGerb
author:JovanGerb
refactor(translate): merge `expand` into `applyReplacementFun` This PR refactors the main translation loop (`applyReplacementFun`) of `to_additive `/`to_dual` so that it operates on free variables instead of loose bound variables. This will make it much easier to implement the reordering of arguments of arguments, which is something we need for `to_dual`. The other loop that was run beforehand, `expand`, was separate because it required free variables instead of loose bound variables, but now it won't make sense anymore to have it be a separate loop, so I've merged it into the `applyReplacementFun` implementation. Ideally, we would want to use `Meta.transform` for this, but unfortunately this isn't good enough, because we need more control over when to do recursive calls. So, we copy/inline the implementation of `Meta.transform`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta 97/78 Mathlib/Tactic/Translate/Core.lean,MathlibTest/toAdditive.lean 2 7 ['JovanGerb', 'eric-wieser', 'github-actions', 'leanprover-radar', 'mathlib4-merge-conflict-bot'] joneugster
assignee:joneugster
0-37338
10 hours ago
0-29528
8 hours ago
21-81684
21 days
33981 eric-wieser
author:eric-wieser
fix: use the tracing API to detect trace options --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) easy t-meta 2/2 Mathlib/Tactic/CC.lean,Mathlib/Tactic/Translate/Core.lean 2 2 ['JovanGerb', 'github-actions'] nobody
0-37232
10 hours ago
0-32937
9 hours ago
0-32757
9 hours
33975 pfaffelh
author:pfaffelh
feat(Data/Set/Dissipate): Introduce dissipate s x := ⋂ y ≤ x, s y Introduce Dissipate s x := ⋂ y ≤ x, s y (Data/Set/Dissipate), which is parallel to Data/Set/Accumulate and provide some API for it. This will be used for compact systems in another PR. Co-authored-by: Rémy Degenne [remydegenne@gmail.com](mailto:remydegenne@gmail.com) This PR continues the work from https://github.com/leanprover-community/mathlib4/pull/25899. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data new-contributor 146/0 Mathlib.lean,Mathlib/Data/Set/Dissipate.lean 2 7 ['github-actions', 'pfaffelh', 'vihdzp'] nobody
0-36860
10 hours ago
0-33704
9 hours ago
0-33524
9 hours
33821 JohnnyTeutonic
author:JohnnyTeutonic
feat(LinearAlgebra/Matrix/Hermitian): add IsSkewHermitian predicate Adds `IsSkewHermitian` predicate for matrices satisfying Aᴴ = -A. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
29/0 Mathlib/LinearAlgebra/Matrix/Hermitian.lean 1 5 ['JohnnyTeutonic', 'github-actions', 'themathqueen'] nobody
0-35970
9 hours ago
4-28861
4 days ago
0-43313
12 hours
33967 wangying11123
author:wangying11123
feat(Analysis/Convex/Between): Add Sbtw_expand and Wbtw_expand Complete the theorems related to between_expand Add four theorems `Wbtw.trans_expand_left` If four points `w x y z`,`Wbtw R w x y`,`Wbtw R x y z` and `x ≠ y`, then `Wbtw R w x z`. `Wbtw.trans_expand_right` If four points `w x y z`,`Wbtw R w x y`,`Wbtw R x y z` and `x ≠ y`, then `Wbtw R w y z`. `Sbtw.trans_expand_left` If four points `w x y z`,`Sbtw R w x y` and `Sbtw R x y z` , then `Sbtw R w x z`. `Sbtw.trans_expand_right` If four points `w x y z`,`Sbtw R w x y` and `Sbtw R x y z` , then `Sbtw R w y z`. t-analysis new-contributor 45/0 Mathlib/Analysis/Convex/Between.lean 1 3 ['eric-wieser', 'github-actions'] nobody
0-35858
9 hours ago
unknown
unknown
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` 157/7 Mathlib/Analysis/Convex/Cone/Basic.lean,Mathlib/Analysis/Convex/Cone/Dual.lean,Mathlib/Analysis/InnerProductSpace/Orthogonal.lean,Mathlib/Topology/Algebra/Module/ClosedSubmodule.lean 4 26 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'sgouezel', 'yoh-tanimoto'] sgouezel
assignee:sgouezel
0-35355
9 hours ago
0-33297
9 hours ago
20-60256
20 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." - [x] depends on: #27261 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology new-contributor 110/0 Mathlib.lean,Mathlib/Topology/FoldTrans.lean 2 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
0-35242
9 hours ago
0-32610
9 hours ago
0-34084
9 hours
33983 erdOne
author:erdOne
feat(AlgebraicGeometry): union of disjoint affine opens is affine --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebraic-geometry 57/2 Mathlib/AlgebraicGeometry/Limits.lean 1 1 ['github-actions'] nobody
0-35006
9 hours ago
0-32541
8 hours ago
0-32361
8 hours
33443 sahanwijetunga
author:sahanwijetunga
feat: Define Isometries of Bilinear Spaces --- We define Isometries of Bilinear Spaces, closely following the implementation of isometries of quadratic spaces. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra new-contributor
label:t-algebra$
275/0 Mathlib.lean,Mathlib/LinearAlgebra/BilinearForm/Isometry.lean,Mathlib/LinearAlgebra/BilinearForm/IsometryEquiv.lean 3 1 ['github-actions'] dagurtomas
assignee:dagurtomas
0-34362
9 hours ago
0-32165
8 hours ago
13-58833
13 days
33607 xgenereux
author:xgenereux
feat: primeSpectrum_eq_of_KrullDimLEOne Given a local ring `R` which is also a domain with `Ring.KrullDimLE 1 R` (or equivalently `Ring.DimensionLEOne`) a prime is either `⊥` or`⊤`. The application I have in mind is `IsDiscreteValuationRing R`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-ring-theory 21/11 Mathlib/Order/BoundedOrder/Basic.lean,Mathlib/Order/KrullDimension.lean,Mathlib/RingTheory/Spectrum/Prime/Topology.lean 3 8 ['erdOne', 'github-actions', 'xgenereux'] alreadydone and mariainesdff
assignee:alreadydone assignee:mariainesdff
0-33427
9 hours ago
0-33427
9 hours ago
5-71503
5 days
32825 erdOne
author:erdOne
perf(RingTheory): `attribute [irreducible] KaehlerDifferential` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-ring-theory 5/1 Mathlib/Algebra/Category/ModuleCat/Differentials/Basic.lean,Mathlib/AlgebraicGeometry/Morphisms/FormallyUnramified.lean,Mathlib/RingTheory/Kaehler/Basic.lean 3 4 ['erdOne', 'github-actions', 'leanprover-radar'] nobody
0-32900
9 hours ago
33-23568
33 days ago
33-23388
33 days
33982 erdOne
author:erdOne
feat(AlgebraicGeometry): being locally artinian is local --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebraic-geometry large-import 133/94 Mathlib/AlgebraicGeometry/Artinian.lean,Mathlib/AlgebraicGeometry/Morphisms/Immersion.lean,Mathlib/AlgebraicGeometry/Noetherian.lean,Mathlib/AlgebraicGeometry/SpreadingOut.lean 4 1 ['github-actions'] nobody
0-32879
9 hours ago
0-31899
8 hours ago
0-31719
8 hours
33941 YellPika
author:YellPika
feat(Order/OmegaCompletePartialOrder): teach fun_prop about ωScottContinuous functions This PR adds the necessary lemmas and attributes for the `fun_prop` tactic with work with `ωScottContinuous` functions. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-order 81/31 Mathlib/Order/OmegaCompletePartialOrder.lean,Mathlib/Order/ScottContinuity.lean 2 1 ['github-actions'] nobody
0-32801
9 hours ago
1-12281
1 day ago
1-12101
1 day
33986 martinwintermath
author:martinwintermath
feat(Order/ModularLattice): add lemmas to construct IsCompl from Disjoint/Codisjoint on complemented modular lattices This PR adds two lemmas to construct `IsCompl` from `Disjoint`/`Codisjoint` on a complemented modular lattices: * `Disjoint.exists_isCompl` enlarges one element of a disjoint pair to obtain a complementary pair. * `Codisjoint.exists_isCompl` shrinks one element of a codisjoint pair to obtain a complementary pair. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-order 17/0 Mathlib/Order/ModularLattice.lean 1 1 ['github-actions'] nobody
0-32796
9 hours ago
0-28561
7 hours ago
0-28381
7 hours
33188 BryceT233
author:BryceT233
feat: MvPowerSeries.rename This file establishes the `rename` operation on multivariate power series under an injective map, which modifies the set of variables. This file is patterned after `MvPolynomials/Rename.lean` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-ring-theory awaiting-author 335/1 Mathlib.lean,Mathlib/Data/Finsupp/Basic.lean,Mathlib/RingTheory/MvPowerSeries/Basic.lean,Mathlib/RingTheory/MvPowerSeries/Rename.lean 4 7 ['BryceT233', 'Komyyy', 'erdOne', 'github-actions'] erdOne
assignee:erdOne
0-32347
8 hours ago
18-58230
18 days ago
4-77241
4 days
33768 vihdzp
author:vihdzp
chore(Order/RelClasses): remove redundant instances --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order 0/20 Mathlib/Order/RelClasses.lean 1 5 ['github-actions', 'leanprover-radar', 'vihdzp'] Vierkantor
assignee:Vierkantor
0-31727
8 hours ago
0-41243
11 hours ago
6-4738
6 days
32534 erdOne
author:erdOne
feat(AlgebraicGeometry): Zariski's main theorem --- - [ ] depends on: #33903 - [ ] depends on: #33805 - [ ] depends on: #33803 - [ ] depends on: #33722 - [ ] depends on: #33718 - [ ] depends on: #32811 - [ ] depends on: #32803 - [ ] depends on: #33535 - [ ] depends on: #33469 - [ ] depends on: #33555 - [x] depends on: #33553 - [x] depends on: #32530 - [x] depends on: #32528 - [x] depends on: #32429 - [x] depends on: #32375 - [x] depends on: #30885 - [x] depends on: #32536 - [x] depends on: #32537 - [x] depends on: #32595 - [x] depends on: #32596 - [x] depends on: #32813 - [x] depends on: #32809 - [x] depends on: #32802 - [x] depends on: #33468 - [x] depends on: #32665 - [x] depends on: #32823 - [x] depends on: #32806 - [x] depends on: #32837 - [x] depends on: #33537 - [x] depends on: #33476 - [x] depends on: #33556 - [x] depends on: #33536 - [x] depends on: #33472 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-ring-theory blocked-by-other-PR 5749/0 Mathlib.lean,Mathlib/AlgebraicGeometry/Morphisms/QuasiFinite.lean,Mathlib/CFT/ActualStuff.lean,Mathlib/CFT/Etale.lean,Mathlib/CFT/EtaleLocalization.lean,Mathlib/CFT/Flat.lean,Mathlib/CFT/IntegralClosure.lean,Mathlib/CFT/IsStandardEtale.lean,Mathlib/CFT/Junk.lean,Mathlib/CFT/NewNo.lean,Mathlib/CFT/No.lean,Mathlib/CFT/Nonsense.lean,Mathlib/CFT/Normalization.lean,Mathlib/CFT/Prestuff.lean,Mathlib/CFT/SeparableResidueStruct.lean,Mathlib/CFT/Smooth.lean,Mathlib/CFT/SmoothFibers.lean,Mathlib/CFT/StandardSmooth.lean,Mathlib/CFT/Stuff.lean,Mathlib/CFT/Stuff2.lean,Mathlib/CFT/ZariskiMain.lean,Mathlib/RingTheory/QuasiFinite.lean,Mathlib/RingTheory/ZariskiMain.lean 23 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
0-31395
8 hours ago
unknown
unknown
33984 erdOne
author:erdOne
feat(AlgebraicGeometry): quasi-finite morphisms --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebraic-geometry 107/0 Mathlib.lean,Mathlib/AlgebraicGeometry/Morphisms/QuasiFinite.lean 2 1 ['github-actions'] nobody
0-31308
8 hours ago
0-29415
8 hours ago
0-29235
8 hours
32027 alreadydone
author:alreadydone
feat(Counterexamples): invertible module not isomorphic to any ideal --- - [x] depends on: #30736 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-ring-theory 95/3 Counterexamples.lean,Counterexamples/InvertibleModuleNotIdeal.lean,Mathlib/Algebra/TrivSqZeroExt.lean,Mathlib/RingTheory/PicardGroup.lean 4 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] chrisflav
assignee:chrisflav
0-31259
8 hours ago
3-57800
3 days ago
3-57620
3 days
33831 vihdzp
author:vihdzp
refactor(RingTheory/Polynomial/SmallDegreeVieta): convert to {p : R[X]} (hp : p.natDegree = 2) Co-authored-by: Christopher Hoskin --- Adopted from #29921. I've applied all pending suggestions. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-ring-theory 112/48 Mathlib/Algebra/Polynomial/Basic.lean,Mathlib/Algebra/Polynomial/Roots.lean,Mathlib/RingTheory/Polynomial/SmallDegreeVieta.lean 3 1 ['github-actions'] chrisflav
assignee:chrisflav
0-31256
8 hours ago
4-29286
4 days ago
4-29106
4 days
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. This allows one to prove two paths are homotopic by transferring to the fundamental groupoid and using `simp`. --- 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). [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebraic-topology new-contributor awaiting-author please-merge-master 6/0 Mathlib/AlgebraicTopology/FundamentalGroupoid/Basic.lean 1 13 ['Sebi-Kumar', 'alreadydone', 'github-actions', 'mathlib4-merge-conflict-bot', 'mattrobball', 'robin-carlier'] mattrobball
assignee:mattrobball
0-31053
8 hours ago
12-77667
12 days ago
3-33381
3 days
33968 edegeltje
author:edegeltje
chore(CategoryTheory/Limits/Shapes/Pullback): Split `CommSq` Split the file `CategoryTheory/Limits/Shapes/Pullback/CommSq.lean` in twain: move defs/thms about `BicartesianSq`, `HasZeroObject` and `HasZeroMorphism` to `CategoryTheory/Limits/Shapes/Pullback/BicartesianSq.lean` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-CI t-category-theory 1626/1545 Mathlib/CategoryTheory/CommSq.lean,Mathlib/CategoryTheory/Limits/Shapes/Opposites/Pullbacks.lean,Mathlib/CategoryTheory/Limits/Shapes/Pullback/CommSq.lean,Mathlib/CategoryTheory/Limits/Shapes/Pullback/IsPullback/Basic.lean,Mathlib/CategoryTheory/Limits/Shapes/Pullback/IsPullback/BicartesianSq.lean,Mathlib/CategoryTheory/Limits/Shapes/Pullback/IsPullback/Defs.lean,Mathlib/CategoryTheory/Limits/Shapes/Pullback/PullbackCone.lean 7 1 ['github-actions'] nobody
0-30845
8 hours ago
unknown
unknown
33985 YellPika
author:YellPika
feat(Order/OmegaCompletePartialOrder): `OmegaCompletePartialOrder` instance for `Sum` with basic `ωScottContinuous` lemmas This PR adds an `OmegaCompletePartialOrder` instance for `Sum`, along with `ωScottContinuous` lemmas for basic operations (`inl`, `inr`, `elim`). Appropriate lemmas are marked with `@[fun_prop]` so that the `fun_prop` tactic can automatically deduce `ωScottContinuous` proofs for functions involving `Sum`s (e.g. see the proof of `Sum.ωScottContinuous_map`). - [ ] depends on: #33941 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor large-import blocked-by-other-PR 330/32 Mathlib/Data/Sum/Order.lean,Mathlib/Order/OmegaCompletePartialOrder.lean,Mathlib/Order/ScottContinuity.lean 3 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
0-30812
8 hours ago
0-33532
9 hours ago
0-6
6 seconds
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) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author new-contributor t-measure-probability 363/0 Mathlib.lean,Mathlib/MeasureTheory/VectorMeasure/Variation/Defs.lean 2 44 ['EtienneC30', 'github-actions', 'mathlib4-merge-conflict-bot', 'sgouezel', 'yoh-tanimoto'] EtienneC30
assignee:EtienneC30
0-30754
8 hours ago
167-64677
167 days ago
30-85938
30 days
33819 bjornsolheim
author:bjornsolheim
feat(Analysis/Convex): diameter of a standard simplex diameter of a standard simplex --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis 48/0 Mathlib/Analysis/Convex/StdSimplex.lean,Mathlib/Topology/MetricSpace/Pseudo/Pi.lean 2 8 ['bjornsolheim', 'github-actions', 'j-loreaux', 'themathqueen'] nobody
0-29504
8 hours ago
0-27763
7 hours ago
3-45916
3 days
32924 chrisflav
author:chrisflav
feat(RingTheory/Smooth): smooth is equivalent to locally standard smooth From Pi1. --- - [x] depends on: #32925 The import increase is expected. The file `Mathlib.RingTheory.Smooth.StandardSmoothOfFree` is a leaf file that was planned to contain this proof. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-ring-theory large-import 265/4 Mathlib.lean,Mathlib/Algebra/Module/FinitePresentation.lean,Mathlib/Algebra/Module/LocalizedModule/Basic.lean,Mathlib/RingTheory/Etale/Basic.lean,Mathlib/RingTheory/Etale/Kaehler.lean,Mathlib/RingTheory/Ideal/Span.lean,Mathlib/RingTheory/Localization/Away/Basic.lean,Mathlib/RingTheory/Localization/Module.lean,Mathlib/RingTheory/RingHom/LocallyStandardSmooth.lean,Mathlib/RingTheory/RingHom/StandardSmooth.lean,Mathlib/RingTheory/Smooth/Basic.lean,Mathlib/RingTheory/Smooth/Locus.lean,Mathlib/RingTheory/Smooth/StandardSmoothOfFree.lean,Mathlib/RingTheory/Support.lean 14 27 ['chrisflav', 'erdOne', 'github-actions', 'mathlib4-dependent-issues-bot'] nobody
0-29153
8 hours ago
0-29153
8 hours ago
3-73584
3 days
32042 chrisflav
author:chrisflav
feat(AlgebraicGeometry): quasi compact covers This will be used to define the fpqc topology on `Scheme`. From Proetale. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebraic-geometry 311/13 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 18 ['chrisflav', 'erdOne', 'github-actions'] joneugster
assignee:joneugster
0-28194
7 hours ago
6-43396
6 days ago
50-62645
50 days
33987 MrQubo
author:MrQubo
doc(Tactic/Lift): Mention `norm_cast` in documentation of `lift` It often makes sense to try `norm_cast` after `lift`. This makes it easier to discover the former. --- [#mathlib4 > RFC: `lift` tactic postprocessing](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/RFC.3A.20.60lift.60.20tactic.20postprocessing/with/568045912) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta new-contributor 2/0 Mathlib/Tactic/Lift.lean 1 1 ['github-actions'] nobody
0-27383
7 hours ago
0-23235
6 hours ago
0-23055
6 hours
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order 395/377 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/RepresentationTheory/Subrepresentation.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 59 46 ['Vierkantor', 'YaelDillies', 'github-actions', 'jcommelin', 'leanprover-bot', 'leanprover-radar', 'mathlib4-merge-conflict-bot', 'plp127', 'vihdzp'] bryangingechen
assignee:bryangingechen
0-27226
7 hours ago
0-27376
7 hours ago
35-68260
35 days
33420 YanYablonovskiy
author:YanYablonovskiy
feat: order types Adding OrderTypes, equivalence classes of linear orders up to order isomorphism. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order new-contributor merge-conflict 440/17 Mathlib.lean,Mathlib/Data/Sum/Order.lean,Mathlib/Order/Category/LinOrd.lean,Mathlib/Order/Defs/LinearOrder.lean,Mathlib/Order/Hom/Basic.lean,Mathlib/Order/Hom/Lex.lean,Mathlib/Order/Types/Basic.lean,Mathlib/Order/Types/Defs.lean 8 135 ['YaelDillies', 'YanYablonovskiy', 'github-actions', 'mathlib4-merge-conflict-bot', 'vihdzp'] nobody
0-26808
7 hours ago
unknown
unknown
33393 grunweg
author:grunweg
chore: extend the whitespace linter to structure and instance fields --- - [ ] depends on: #30658 - [x] depends on: #33747 This will require a large number of fixes: land these changes separately (but doing so is nice!). [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) please-adopt merge-conflict large-import blocked-by-other-PR 2202/595 Archive/Imo/Imo2010Q5.lean,Archive/Wiedijk100Theorems/BuffonsNeedle.lean,Counterexamples/CliffordAlgebraNotInjective.lean,Mathlib/Algebra/AffineMonoid/Basic.lean,Mathlib/Algebra/Algebra/Defs.lean,Mathlib/Algebra/Algebra/Subalgebra/Basic.lean,Mathlib/Algebra/Category/Grp/Basic.lean,Mathlib/Algebra/Category/Grp/EpiMono.lean,Mathlib/Algebra/Category/ModuleCat/ChangeOfRings.lean,Mathlib/Algebra/Category/ModuleCat/Presheaf.lean,Mathlib/Algebra/Category/ModuleCat/Topology/Basic.lean,Mathlib/Algebra/Category/MonCat/Limits.lean,Mathlib/Algebra/DirectSum/Ring.lean,Mathlib/Algebra/Group/AddChar.lean,Mathlib/Algebra/Group/Hom/Basic.lean,Mathlib/Algebra/Group/Submonoid/Operations.lean,Mathlib/Algebra/GroupWithZero/WithZero.lean,Mathlib/Algebra/Lie/Abelian.lean,Mathlib/Algebra/Module/Submodule/Defs.lean,Mathlib/Algebra/Module/TransferInstance.lean,Mathlib/Algebra/Order/CauSeq/Basic.lean,Mathlib/Algebra/Order/Monoid/Unbundled/WithTop.lean,Mathlib/Algebra/Order/Nonneg/Ring.lean,Mathlib/Algebra/Order/Ring/WithTop.lean,Mathlib/Algebra/Polynomial/Derivation.lean,Mathlib/Algebra/Polynomial/RuleOfSigns.lean,Mathlib/Algebra/Polynomial/Taylor.lean,Mathlib/Algebra/Quaternion.lean,Mathlib/Algebra/Ring/SumsOfSquares.lean,Mathlib/Algebra/SkewMonoidAlgebra/Basic.lean,Mathlib/Algebra/SkewMonoidAlgebra/Lift.lean,Mathlib/Algebra/Star/StarAlgHom.lean,Mathlib/Algebra/Star/StarRingHom.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Jacobian/Basic.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Projective/Basic.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Projective/Formula.lean,Mathlib/AlgebraicTopology/SimplicialSet/CompStructTruncated.lean,Mathlib/AlgebraicTopology/SimplicialSet/HoFunctorMonoidal.lean,Mathlib/AlgebraicTopology/SimplicialSet/Path.lean,Mathlib/AlgebraicTopology/SimplicialSet/StrictSegal.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Unital.lean,Mathlib/Analysis/Normed/Algebra/Spectrum.lean,Mathlib/Analysis/Normed/Group/SemiNormedGrp/Kernels.lean,Mathlib/Analysis/Normed/Ring/Lemmas.lean,Mathlib/Analysis/Normed/Unbundled/AlgebraNorm.lean,Mathlib/Analysis/Normed/Unbundled/InvariantExtension.lean,Mathlib/Analysis/Normed/Unbundled/RingSeminorm.lean,Mathlib/Analysis/Normed/Unbundled/SeminormFromBounded.lean,Mathlib/Analysis/Normed/Unbundled/SeminormFromConst.lean,Mathlib/Analysis/Normed/Unbundled/SmoothingSeminorm.lean,Mathlib/Analysis/Normed/Unbundled/SpectralNorm.lean,Mathlib/Analysis/ODE/PicardLindelof.lean,Mathlib/Analysis/Real/Pi/Bounds.lean,Mathlib/CategoryTheory/Adjunction/Basic.lean,Mathlib/CategoryTheory/Adjunction/Evaluation.lean,Mathlib/CategoryTheory/Bicategory/Free.lean,Mathlib/CategoryTheory/Functor/Currying.lean,Mathlib/CategoryTheory/Functor/KanExtension/Basic.lean,Mathlib/CategoryTheory/Functor/KanExtension/Dense.lean,Mathlib/CategoryTheory/Generator/Presheaf.lean,Mathlib/CategoryTheory/Limits/Fubini.lean,Mathlib/CategoryTheory/Limits/Preserves/Basic.lean,Mathlib/CategoryTheory/Limits/Preserves/Bifunctor.lean,Mathlib/CategoryTheory/Limits/Preserves/FunctorCategory.lean,Mathlib/CategoryTheory/Limits/Shapes/BinaryProducts.lean,Mathlib/CategoryTheory/Limits/Shapes/Equalizers.lean,Mathlib/CategoryTheory/Limits/Shapes/Images.lean,Mathlib/CategoryTheory/Limits/Shapes/Pullback/Categorical/CatCospanTransform.lean,Mathlib/CategoryTheory/Limits/Types/Coproducts.lean,Mathlib/CategoryTheory/Limits/Types/Products.lean,Mathlib/CategoryTheory/Monad/Comonadicity.lean,Mathlib/CategoryTheory/Monad/Monadicity.lean,Mathlib/CategoryTheory/Monoidal/Action/Basic.lean,Mathlib/CategoryTheory/Monoidal/Action/End.lean,Mathlib/CategoryTheory/Monoidal/Cartesian/CommGrp_.lean,Mathlib/CategoryTheory/Monoidal/Cartesian/Grp_.lean,Mathlib/CategoryTheory/Monoidal/Center.lean,Mathlib/CategoryTheory/Monoidal/Closed/Ideal.lean,Mathlib/CategoryTheory/Monoidal/DayConvolution.lean,Mathlib/CategoryTheory/Monoidal/Mon_.lean,Mathlib/CategoryTheory/Monoidal/OfHasFiniteProducts.lean,Mathlib/CategoryTheory/Monoidal/Opposite.lean,Mathlib/CategoryTheory/MorphismProperty/Limits.lean,Mathlib/CategoryTheory/Opposites.lean,Mathlib/CategoryTheory/Presentable/Directed.lean,Mathlib/CategoryTheory/Sites/CartesianMonoidal.lean,Mathlib/CategoryTheory/Sites/Coherent/ExtensiveColimits.lean,Mathlib/CategoryTheory/Triangulated/Opposite/OpOp.lean,Mathlib/CategoryTheory/WithTerminal/Basic.lean,Mathlib/Combinatorics/SetFamily/LYM.lean,Mathlib/Combinatorics/SimpleGraph/Clique.lean,Mathlib/Computability/AkraBazzi/AkraBazzi.lean,Mathlib/Computability/ContextFreeGrammar.lean,Mathlib/Computability/Language.lean,Mathlib/Computability/Partrec.lean,Mathlib/Computability/PartrecCode.lean,Mathlib/Data/DFinsupp/Notation.lean,Mathlib/Data/ENNReal/Basic.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/Data/EReal/Operations.lean 188 9 ['github-actions', 'grunweg', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
0-24506
6 hours ago
unknown
unknown
33539 BryceT233
author:BryceT233
feat(RingTheory/MvPolynomial): powers of ideal of variables 1. Added a new file `Mathlib/Algebra/Group/Pointwise/Set/Finsupp.lean` for results about pointwise operations on sets and finitely supported functions 2. Provided more APIs for `MvPolynomial.restrictSupport` and defined `restrictSupportIdeal` to be the ideal determined by `restrictSupport R s` when `s` is an upper set 3. Defined `MvPolynomial.idealOfVars` to be the ideal spanned by all variables in `MvPolynomial` and provided results about its powers 4. Provided some helper results while golfing --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author large-import t-ring-theory new-contributor 250/2 Mathlib.lean,Mathlib/Algebra/Group/Pointwise/Set/Basic.lean,Mathlib/Algebra/Group/Pointwise/Set/Finsupp.lean,Mathlib/Algebra/Group/TypeTags/Pointwise.lean,Mathlib/Data/Finsupp/Weight.lean,Mathlib/RingTheory/MvPolynomial/Basic.lean,Mathlib/RingTheory/MvPolynomial/Ideal.lean 7 19 ['BryceT233', 'erdOne', 'github-actions', 'vihdzp'] erdOne
assignee:erdOne
0-23707
6 hours ago
4-54292
4 days ago
6-9529
6 days
33680 BoltonBailey
author:BoltonBailey
feat(Probability/ProbabilityMassFunction): add Total Variation distance Adds the statistical distance/total variation distance. This PR was authored with the support of Claude opus 4.5 --- Note: Perhaps a good thing to do before this PR would be to change the return type of the funlike instance for PMF into a (subtype of) the reals, see #33689, or at least provide an API for that function. Zulip https://leanprover.zulipchat.com/#narrow/channel/217875-Is-there-code-for-X.3F/topic/total.20variation.20distance.20between.20two.20PMFs [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-measure-probability 47/0 Mathlib/Probability/ProbabilityMassFunction/Distance.lean 1 1 ['github-actions'] nobody
0-22515
6 hours ago
unknown
unknown
33942 artie2000
author:artie2000
refactor: unbundle `GroupCone` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-algebra
label:t-algebra$
192/10 Mathlib/Algebra/Group/Subgroup/Defs.lean,Mathlib/Algebra/Group/Submonoid/Support.lean,Mathlib/Algebra/Order/Group/Cone.lean,Mathlib/Tactic/Translate/ToAdditive.lean 4 3 ['artie2000', 'github-actions', 'vihdzp'] nobody
0-22412
6 hours ago
unknown
unknown
33944 artie2000
author:artie2000
feat: formally real rings --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra awaiting-author
label:t-algebra$
100/0 Mathlib.lean,Mathlib/Algebra/Ring/IsFormallyReal.lean,Mathlib/Algebra/Ring/SumsOfSquares.lean 3 15 ['artie2000', 'github-actions', 'vihdzp'] nobody
0-22256
6 hours ago
unknown
unknown
33817 FlAmmmmING
author:FlAmmmmING
fix(Combinatorics/Enumerative/Schroder.lean): Fix the definition and theorem of smallSchroder. In the previous definition, the small Schröder numbers were defined as ```LaTeX s_0 = 1, s_1 = 1, s_2 = 1, s_3 = 3... ``` , which does not match the sequence listed in OEIS A006318. Moreover, this definition makes it difficult to correctly write the generating function for the small Schröder numbers. This PR fixes this issue. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-combinatorics large-import 47/39 Mathlib/Combinatorics/Enumerative/Schroder.lean 1 19 ['FlAmmmmING', 'github-actions', 'vihdzp'] nobody
0-20742
5 hours ago
0-19599
5 hours ago
4-50003
4 days
33752 mcdoll
author:mcdoll
feat(Analysis/FourierSchwartz): the derivative of the Fourier transform Calculate the derivative (`fderiv` and `lineDerivOp`) of the (inverse) Fourier transform. We also generalize `evalCLM` slightly and make it's arguments explicit. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis 140/9 Mathlib/Analysis/Distribution/FourierSchwartz.lean,Mathlib/Analysis/Distribution/SchwartzSpace.lean,Mathlib/Analysis/Distribution/TemperateGrowth.lean 3 6 ['github-actions', 'mcdoll', 'sgouezel'] sgouezel
assignee:sgouezel
0-20316
5 hours ago
0-19420
5 hours ago
5-66022
5 days
33411 IlPreteRosso
author:IlPreteRosso
feat(Analysis/DiscreteConvolution): Discrete convolution API basics This is the first PR is a series of PRs towards the proposed API and ℓ1 Banach algebra. Defines discrete convolution of functions `f : M → E` and `g : M → E'` over a monoid `M` using a bilinear map `L : E →ₗ[S] E' →ₗ[S] F`: `(f ⋆[L] g) x = ∑' (a, b) : mulFiber x, L (f a) (g b)` where `abbrev mulFiber (x : M) : Set (M × M) := Set.mulAntidiagonal Set.univ Set.univ x` t-analysis new-contributor 968/11 Mathlib.lean,Mathlib/Algebra/BigOperators/CauchyProduct.lean,Mathlib/Algebra/Order/Antidiag/Prod.lean,Mathlib/Topology/Algebra/InfiniteSum/DiscreteConvolution.lean 4 25 ['IlPreteRosso', 'github-actions', 'j-loreaux', 'plp127'] urkud
assignee:urkud
0-16863
4 hours ago
0-15753
4 hours ago
13-2048
13 days
32851 tdwag123
author:tdwag123
feat(MeasureTheory/Measure/TypeClass/NoAtoms) add `exists_accPt_of_noAtoms` feat(MeasureTheory/Measure/TypeClass/NoAtoms): Added a theorem that states If a set has positive measure under an atomless measure, then it has an accumulation point. Added a lemma in (Topology/DiscreteSubset): If a subset of a topological space has no accumulation points, then it carries the discrete topology. Theorem added: `exists_accPt_of_pos_hausdorffMeasure` Lemma added: `discreteTopology_of_noAccPts ` **Harmonic's Aristotle gave the initial version of the proofs.** I did substantial work shortening the proof from 40 lines and refactoring it into another Lemma. Special thanks to @plp127 and @CoolRmal for the useful feedback in the PR process. **Co-authored-by: @Aristotle-Harmonic ** `---` [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-measure-probability awaiting-author 23/1 Mathlib/MeasureTheory/Measure/Typeclasses/NoAtoms.lean,Mathlib/Topology/DiscreteSubset.lean 2 27 ['CoolRmal', 'Vilin97', 'github-actions', 'plp127', 'sgouezel', 'tdwag123'] urkud
assignee:urkud
0-13391
3 hours ago
12-68431
12 days ago
15-48177
15 days
33873 YaelDillies
author:YaelDillies
chore(Algebra): replace `NoZeroSMulDivisors` with `Module.IsTorsionFree`, losing generality `NoZeroSMulDivisors R M` is mathematically wrong when `R` isn't a domain, so we replace it with the better definition `Module.IsTorsionFree R M` whenever they are equivalent. This PR continues #30563, replacing `NoZeroSMulDivisors R M` with `Module.IsTorsionFree R M` even when this loses generality. --- - [x] depends on: #30563 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra large-import
label:t-algebra$
241/503 Mathlib/Algebra/Algebra/Basic.lean,Mathlib/Algebra/Algebra/NonUnitalSubalgebra.lean,Mathlib/Algebra/Algebra/Subalgebra/Basic.lean,Mathlib/Algebra/Algebra/Tower.lean,Mathlib/Algebra/BigOperators/Finprod.lean,Mathlib/Algebra/Central/Basic.lean,Mathlib/Algebra/GroupWithZero/Action/Pointwise/Finset.lean,Mathlib/Algebra/GroupWithZero/Action/Pointwise/Set.lean,Mathlib/Algebra/GroupWithZero/NonZeroDivisors.lean,Mathlib/Algebra/Module/Basic.lean,Mathlib/Algebra/Module/LinearMap/Basic.lean,Mathlib/Algebra/Module/LinearMap/End.lean,Mathlib/Algebra/Module/LocalizedModule/Basic.lean,Mathlib/Algebra/Module/Submodule/Basic.lean,Mathlib/Algebra/Module/Submodule/Union.lean,Mathlib/Algebra/Module/Torsion/Basic.lean,Mathlib/Algebra/Module/Torsion/Free.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/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/Convex/Strict.lean,Mathlib/Analysis/SpecificLimits/Normed.lean,Mathlib/Data/ENNReal/Action.lean,Mathlib/Data/Finsupp/SMul.lean,Mathlib/FieldTheory/Galois/IsGaloisGroup.lean,Mathlib/Geometry/Euclidean/Triangle.lean,Mathlib/LinearAlgebra/AffineSpace/Slope.lean,Mathlib/LinearAlgebra/Basis/Basic.lean,Mathlib/LinearAlgebra/Eigenspace/Minpoly.lean,Mathlib/LinearAlgebra/LinearIndependent/Lemmas.lean,Mathlib/LinearAlgebra/Multilinear/Basic.lean,Mathlib/LinearAlgebra/Reflection.lean,Mathlib/LinearAlgebra/StdBasis.lean,Mathlib/MeasureTheory/Function/EssSup.lean,Mathlib/MeasureTheory/Function/LpSeminorm/Basic.lean,Mathlib/MeasureTheory/Measure/AEMeasurable.lean,Mathlib/MeasureTheory/Measure/Decomposition/IntegralRNDeriv.lean,Mathlib/MeasureTheory/Measure/Haar/Disintegration.lean,Mathlib/MeasureTheory/Measure/Hausdorff.lean,Mathlib/MeasureTheory/Measure/Map.lean,Mathlib/MeasureTheory/Measure/MeasureSpace.lean,Mathlib/MeasureTheory/OuterMeasure/Induced.lean,Mathlib/RingTheory/Algebraic/Integral.lean,Mathlib/RingTheory/HahnSeries/Lex.lean,Mathlib/RingTheory/HahnSeries/Multiplication.lean,Mathlib/RingTheory/IntegralClosure/IntegralRestrict.lean,Mathlib/RingTheory/IntegralClosure/IsIntegralClosure/Basic.lean,Mathlib/RingTheory/Nilpotent/Basic.lean,Mathlib/RingTheory/NormalClosure.lean,Mathlib/RingTheory/Polynomial/Eisenstein/IsIntegral.lean,Mathlib/RingTheory/QuasiFinite/Basic.lean,Mathlib/RingTheory/TensorProduct/Basic.lean 68 16 ['YaelDillies', 'github-actions', 'jcommelin', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
0-7114
1 hour ago
1-43850
1 day ago
0-2475
41 minutes
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-data large-import 141/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 12 ['Ruben-VandeVelde', 'YaelDillies', 'github-actions', 'mathlib4-merge-conflict-bot'] bryangingechen
assignee:bryangingechen
0-7003
1 hour ago
unknown
unknown
33972 YuvalFilmus
author:YuvalFilmus
feat(Analysis/Polynomial/Order): polynomial has fixed sign beyond largest root We prove that a polynomial has fixed sign beyond its largest root. One could also prove similar results about the smallest root, but they will be more awkward since they will depend on the parity of the (natural) degree; suggestions welcome (perhaps for a future PR). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis 73/0 Mathlib.lean,Mathlib/Analysis/Polynomial/Order.lean 2 6 ['YuvalFilmus', 'github-actions', 'vihdzp'] nobody
0-6529
1 hour ago
0-37198
10 hours ago
0-6812
1 hour
33461 loefflerd
author:loefflerd
feat(NumberTheory/Modular): stabilizers for action on upper halfplane --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP 300/47 Mathlib.lean,Mathlib/Analysis/Complex/UpperHalfPlane/MoebiusAction.lean,Mathlib/Analysis/Complex/UpperHalfPlane/ProjLine.lean,Mathlib/Analysis/Complex/UpperHalfPlane/Topology.lean,Mathlib/LinearAlgebra/Matrix/GeneralLinearGroup/Defs.lean,Mathlib/LinearAlgebra/Matrix/SpecialLinearGroup.lean,Mathlib/NumberTheory/Modular.lean,Mathlib/NumberTheory/ModularForms/Basic.lean 8 1 ['github-actions'] nobody
0-6472
1 hour ago
unknown
unknown
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-computability awaiting-author 57/3 Mathlib/Computability/Encoding.lean,Mathlib/Data/List/Basic.lean,Mathlib/Data/Sum/Basic.lean 3 11 ['BoltonBailey', 'MichaelStollBayreuth', 'YaelDillies', 'github-actions'] YaelDillies
assignee:YaelDillies
0-5649
1 hour ago
0-5649
1 hour ago
43-4541
43 days
33291 BoltonBailey
author:BoltonBailey
refactor(Computability): file for state transition systems This PR makes a new file to contain content having to do with state transition systems defined by a function `σ → Option σ`. This content was previously split over `PostTuringMachine.lean` and `TMComputable.lean`, but since these definitions don't only apply to Turing machines in particular, it seems sensible to refactor them and remove them from the `Turing` namespace and put them in a new `StateTransition` namespace. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-computability 320/233 Mathlib.lean,Mathlib/Computability/PostTuringMachine.lean,Mathlib/Computability/StateTransition.lean,Mathlib/Computability/TMConfig.lean,Mathlib/Computability/TMToPartrec.lean,Mathlib/Computability/TuringMachine.lean 6 5 ['YaelDillies', 'github-actions'] YaelDillies
assignee:YaelDillies
0-5285
1 hour ago
0-5295
1 hour ago
20-15565
20 days
33989 xroblot
author:xroblot
feat: elements of `adjoin S` are fixed by `m` iff elements of `S` are This PR proves: ```lean (∀ x ∈ adjoin F S, m • x = x) ↔ (∀ x ∈ S, m • x = x) ``` both in the `Algebra.adjoin` and `IntermediateField.adjoin` cases --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
23/0 Mathlib/Algebra/MvPolynomial/Eval.lean,Mathlib/FieldTheory/IntermediateField/Adjoin/Basic.lean 2 1 ['github-actions'] nobody
0-4600
1 hour ago
unknown
unknown
33895 jessealama
author:jessealama
feat(Computability/Primrec): add list_take, list_drop, list_modify, and list_set This PR shows that several list operations from Lean core are primitive recursive: - `list_take`: [`List.take`](https://github.com/leanprover/lean4/blob/master/src/Init/Data/List/TakeDrop.lean) - `list_drop`: [`List.drop`](https://github.com/leanprover/lean4/blob/master/src/Init/Data/List/TakeDrop.lean) - `list_modifyHead'`: [`List.modifyHead`](https://github.com/leanprover/lean4/blob/master/src/Init/Data/List/Nat/Modify.lean) with external data - `list_modify'`: [`List.modify`](https://github.com/leanprover/lean4/blob/master/src/Init/Data/List/Nat/Modify.lean) with external data - `list_modify`: [`List.modify`](https://github.com/leanprover/lean4/blob/master/src/Init/Data/List/Nat/Modify.lean) - `list_set`: [`List.set`](https://github.com/leanprover/lean4/blob/master/src/Init/Prelude.lean) The primed versions (`list_modify'`, `list_modifyHead'`) take a function `g : β → α → α` that depends on external data of type `β`. This generalization enables deriving the other operations: - `list_modify` specializes `list_modify'` with `β = Unit` - `list_set` uses `list_modify'` via `List.set_eq_modify` new-contributor t-computability 67/4 Mathlib/Computability/Primrec/List.lean 1 1 ['github-actions'] nobody
0-4092
1 hour ago
0-3238
50 minutes ago
0-3371
56 minutes
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. --- - [ ] depends on: #33956 - [ ] depends on: #33955 - [x] depends on: #33084 - [x] depends on: #33085 - [x] depends on: #33086 - [ ] depends on: #33087 - [ ] depends on: #33088 - [x] depends on: #26171 - [x] depends on: #26166 - [x] depends on: #26365 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebraic-topology WIP t-category-theory blocked-by-other-PR 1531/2 Mathlib.lean,Mathlib/AlgebraicTopology/ModelCategory/Bifibrant.lean,Mathlib/AlgebraicTopology/ModelCategory/BifibrantObjectHomotopy.lean,Mathlib/AlgebraicTopology/ModelCategory/CofibrantObjectHomotopy.lean,Mathlib/AlgebraicTopology/ModelCategory/DerivabilityStructureCofibrant.lean,Mathlib/AlgebraicTopology/ModelCategory/DerivabilityStructureFibrant.lean,Mathlib/AlgebraicTopology/ModelCategory/FibrantObjectHomotopy.lean,Mathlib/AlgebraicTopology/ModelCategory/FundamentalLemma.lean,Mathlib/AlgebraicTopology/ModelCategory/Homotopy.lean,Mathlib/AlgebraicTopology/ModelCategory/IsCofibrant.lean,Mathlib/CategoryTheory/Localization/LocalizerMorphism.lean 11 4 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
0-4036
1 hour ago
unknown
unknown
30658 grunweg
author:grunweg
feat: extend the `whitespace` linter to proof bodies --- - [x] depends on: #30663 - [x] depends on: #30685 - [x] depends on: #30687 - [x] depends on: #30688 - [x] depends on: #30689 - [x] depends on: #30691 - [x] depends on: #30723 - [x] depends on: #30724 - [x] depends on: #30725 - [x] depends on: leanprover/lean4#11780 - [ ] depends on: leanprover/lean4#12006 - [ ] depends on: leanprover/lean4#11686 - [x] depends on: #33705 - [x] depends on: #33706 - [x] depends on: #33716 - [x] depends on: #33234 - [x] depends on: #33342 - [x] depends on: #33708 - [x] depends on: #33758 - [x] depends on: #33759 - [x] depends on: #33789 - [ ] depends on: #33815 - [x] depends on: #33816 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR large-import awaiting-CI t-linter 2021/467 Archive/Imo/Imo2010Q5.lean,Archive/Wiedijk100Theorems/BuffonsNeedle.lean,Counterexamples/CliffordAlgebraNotInjective.lean,Mathlib/Algebra/AffineMonoid/Basic.lean,Mathlib/Algebra/Category/Grp/EpiMono.lean,Mathlib/Algebra/Module/TransferInstance.lean,Mathlib/Algebra/Order/CauSeq/Basic.lean,Mathlib/Algebra/Polynomial/RuleOfSigns.lean,Mathlib/Algebra/Quaternion.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Jacobian/Basic.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Projective/Basic.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Projective/Formula.lean,Mathlib/AlgebraicTopology/SimplicialSet/CompStructTruncated.lean,Mathlib/AlgebraicTopology/SimplicialSet/Path.lean,Mathlib/AlgebraicTopology/SimplicialSet/StrictSegal.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Unital.lean,Mathlib/Analysis/Normed/Algebra/Spectrum.lean,Mathlib/Analysis/ODE/PicardLindelof.lean,Mathlib/Analysis/Real/Pi/Bounds.lean,Mathlib/CategoryTheory/Comma/Over/OverClass.lean,Mathlib/CategoryTheory/Limits/Shapes/BinaryProducts.lean,Mathlib/CategoryTheory/Monoidal/Action/Basic.lean,Mathlib/CategoryTheory/Monoidal/Cartesian/CommGrp_.lean,Mathlib/CategoryTheory/Monoidal/Mon_.lean,Mathlib/CategoryTheory/Monoidal/OfHasFiniteProducts.lean,Mathlib/Combinatorics/SetFamily/LYM.lean,Mathlib/Computability/AkraBazzi/AkraBazzi.lean,Mathlib/Computability/ContextFreeGrammar.lean,Mathlib/Computability/Language.lean,Mathlib/Computability/Partrec.lean,Mathlib/Computability/PartrecCode.lean,Mathlib/Data/DFinsupp/Notation.lean,Mathlib/Data/ENNReal/Basic.lean,Mathlib/Data/EReal/Operations.lean,Mathlib/Data/Fin/Fin2.lean,Mathlib/Data/Finset/Slice.lean,Mathlib/Data/Finset/Sort.lean,Mathlib/Data/Finsupp/Notation.lean,Mathlib/Data/Matrix/Cartan.lean,Mathlib/Data/NNReal/Defs.lean,Mathlib/Data/Num/Bitwise.lean,Mathlib/Data/PNat/Xgcd.lean,Mathlib/Data/Sym/Sym2.lean,Mathlib/Data/Vector/MapLemmas.lean,Mathlib/FieldTheory/CardinalEmb.lean,Mathlib/FieldTheory/Finite/Extension.lean,Mathlib/FieldTheory/Laurent.lean,Mathlib/Geometry/Manifold/Notation.lean,Mathlib/GroupTheory/FreeGroup/Reduce.lean,Mathlib/LinearAlgebra/TensorPower/Symmetric.lean,Mathlib/LinearAlgebra/TensorProduct/Basic.lean,Mathlib/MeasureTheory/Function/ConditionalExpectation/PullOut.lean,Mathlib/MeasureTheory/Integral/TorusIntegral.lean,Mathlib/ModelTheory/Syntax.lean,Mathlib/NumberTheory/Niven.lean,Mathlib/Probability/CondVar.lean,Mathlib/Probability/Independence/Conditional.lean,Mathlib/RingTheory/Nilpotent/Exp.lean,Mathlib/Tactic/Linter/DirectoryDependency.lean,Mathlib/Tactic/Linter/Whitespace.lean,Mathlib/Tactic/Ring/NamePolyVars.lean,Mathlib/Topology/Algebra/IsUniformGroup/Defs.lean,Mathlib/Topology/Category/TopCat/Limits/Basic.lean,Mathlib/Topology/Instances/Rat.lean,Mathlib/Util/Superscript.lean,MathlibTest/WhitespaceLinter.lean 66 52 ['SnirBroshi', 'adomani', 'github-actions', 'grunweg', 'leanprover-radar', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
0-3835
1 hour ago
unknown
unknown
33904 alreadydone
author:alreadydone
refactor(Algebra): weaken NormalizationMonoid The vast majority of API continue to hold under this weakened notion of NormalizationMonoid; only a handful requires the original notion, which is renamed StrongNormalizationMonoid. Every monoid admits a weakened NormalizationMonoid structure, and every GCDMonoid admits a weakened NormalizedGCDMonoid structure. This allows us to generalize [Polynomial.normalizedGcdMonoid](https://leanprover-community.github.io/mathlib4_docs/Mathlib/RingTheory/Polynomial/Content.html#Polynomial.normalizedGcdMonoid) to all GCDMonoids. --- - [ ] depends on: #33851 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-ring-theory t-algebra blocked-by-other-PR WIP
label:t-algebra$
845/680 Mathlib/Algebra/BigOperators/Associated.lean,Mathlib/Algebra/GCDMonoid/Basic.lean,Mathlib/Algebra/GCDMonoid/Finset.lean,Mathlib/Algebra/GCDMonoid/FinsetLemmas.lean,Mathlib/Algebra/GCDMonoid/IntegrallyClosed.lean,Mathlib/Algebra/GCDMonoid/Multiset.lean,Mathlib/Algebra/GCDMonoid/Nat.lean,Mathlib/Algebra/GCDMonoid/PUnit.lean,Mathlib/Algebra/GroupWithZero/Action/Faithful.lean,Mathlib/Algebra/GroupWithZero/Action/Opposite.lean,Mathlib/Algebra/GroupWithZero/Associated.lean,Mathlib/Algebra/GroupWithZero/Basic.lean,Mathlib/Algebra/GroupWithZero/Defs.lean,Mathlib/Algebra/GroupWithZero/Divisibility.lean,Mathlib/Algebra/GroupWithZero/Idempotent.lean,Mathlib/Algebra/GroupWithZero/InjSurj.lean,Mathlib/Algebra/GroupWithZero/Nat.lean,Mathlib/Algebra/GroupWithZero/Submonoid/Primal.lean,Mathlib/Algebra/GroupWithZero/Torsion.lean,Mathlib/Algebra/GroupWithZero/Units/Basic.lean,Mathlib/Algebra/Order/GroupWithZero/Synonym.lean,Mathlib/Algebra/Order/GroupWithZero/Unbundled/Basic.lean,Mathlib/Algebra/Order/Interval/Set/Instances.lean,Mathlib/Algebra/Order/Monoid/Associated.lean,Mathlib/Algebra/Polynomial/FieldDivision.lean,Mathlib/Algebra/Prime/Defs.lean,Mathlib/Algebra/Prime/Lemmas.lean,Mathlib/Algebra/Regular/Basic.lean,Mathlib/Algebra/Ring/Basic.lean,Mathlib/Algebra/Ring/CharZero.lean,Mathlib/Algebra/Ring/Divisibility/Lemmas.lean,Mathlib/Algebra/Ring/Int/Defs.lean,Mathlib/Algebra/Ring/NonZeroDivisors.lean,Mathlib/Algebra/Ring/PUnit.lean,Mathlib/Algebra/Ring/Rat.lean,Mathlib/Algebra/Ring/Regular.lean,Mathlib/Algebra/Squarefree/Basic.lean,Mathlib/Analysis/Meromorphic/TrailingCoefficient.lean,Mathlib/Analysis/Normed/Field/UnitBall.lean,Mathlib/Combinatorics/Additive/AP/Three/Defs.lean,Mathlib/Data/List/Prime.lean,Mathlib/Data/Matrix/Basic.lean,Mathlib/Data/Matrix/Composition.lean,Mathlib/LinearAlgebra/Eigenspace/Semisimple.lean,Mathlib/NumberTheory/FLT/Basic.lean,Mathlib/RingTheory/ChainOfDivisors.lean,Mathlib/RingTheory/DedekindDomain/Ideal/Basic.lean,Mathlib/RingTheory/DedekindDomain/Ideal/Lemmas.lean,Mathlib/RingTheory/DiscreteValuationRing/Basic.lean,Mathlib/RingTheory/IntegralDomain.lean,Mathlib/RingTheory/Multiplicity.lean,Mathlib/RingTheory/Nilpotent/Basic.lean,Mathlib/RingTheory/OreLocalization/OreSet.lean,Mathlib/RingTheory/Polynomial/Content.lean,Mathlib/RingTheory/Polynomial/ContentIdeal.lean,Mathlib/RingTheory/Polynomial/Eisenstein/IsIntegral.lean,Mathlib/RingTheory/Polynomial/GaussLemma.lean,Mathlib/RingTheory/Polynomial/Nilpotent.lean,Mathlib/RingTheory/Polynomial/UniqueFactorization.lean,Mathlib/RingTheory/PowerSeries/Inverse.lean,Mathlib/RingTheory/Prime.lean,Mathlib/RingTheory/PrincipalIdealDomain.lean,Mathlib/RingTheory/Radical.lean,Mathlib/RingTheory/RootsOfUnity/PrimitiveRoots.lean,Mathlib/RingTheory/Spectrum/Prime/Polynomial.lean,Mathlib/RingTheory/UniqueFactorizationDomain/Basic.lean,Mathlib/RingTheory/UniqueFactorizationDomain/Defs.lean,Mathlib/RingTheory/UniqueFactorizationDomain/FactorSet.lean,Mathlib/RingTheory/UniqueFactorizationDomain/Finite.lean,Mathlib/RingTheory/UniqueFactorizationDomain/Finsupp.lean,Mathlib/RingTheory/UniqueFactorizationDomain/GCDMonoid.lean,Mathlib/RingTheory/UniqueFactorizationDomain/Ideal.lean,Mathlib/RingTheory/UniqueFactorizationDomain/Multiplicative.lean,Mathlib/RingTheory/UniqueFactorizationDomain/Multiplicity.lean,Mathlib/RingTheory/UniqueFactorizationDomain/NormalizedFactors.lean,Mathlib/SetTheory/Nimber/Field.lean,Mathlib/Tactic/FieldSimp/Lemmas.lean,MathlibTest/grind/panic.lean 78 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
0-3583
59 minutes ago
unknown
unknown
33909 YaelDillies
author:YaelDillies
feat(SetTheory/Cardinal): more lemmas about `ENat` and deduplicate a few pairs. From ProofBench --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-set-theory 79/49 Mathlib/Data/Finite/Card.lean,Mathlib/Data/Set/Card.lean,Mathlib/FieldTheory/CardinalEmb.lean,Mathlib/LinearAlgebra/Matrix/Rank.lean,Mathlib/RingTheory/Length.lean,Mathlib/SetTheory/Cardinal/ENat.lean,Mathlib/SetTheory/Cardinal/Finite.lean,Mathlib/SetTheory/Cardinal/NatCount.lean,Mathlib/SetTheory/Cardinal/ToNat.lean 9 2 ['github-actions', 'vihdzp'] nobody
0-2935
48 minutes 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 - [x] depends on: #31908 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics t-measure-probability 158/0 Mathlib.lean,Mathlib/Probability/Combinatorics/BinomialRandomGraph/Defs.lean,Mathlib/Probability/Combinatorics/README.md 3 14 ['DavidLedvinka', 'LibertasSpZ', 'YaelDillies', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] EtienneC30
assignee:EtienneC30
0-2834
47 minutes ago
0-1994
30 minutes ago
34-25038
34 days
32030 newell
author:newell
feat(Analysis/AperiodicOrder/Delone): Delone Sets --- Initial definitions and lemmas for Delone Sets. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis awaiting-author large-import 192/4 Mathlib.lean,Mathlib/Analysis/AperiodicOrder/Delone/Basic.lean,Mathlib/Topology/MetricSpace/Cover.lean,Mathlib/Topology/MetricSpace/MetricSeparated.lean 4 66 ['YaelDillies', 'github-actions', 'j-loreaux', 'newell', 'sgouezel'] j-loreaux
assignee:j-loreaux
0-2438
40 minutes ago
4-86215
4 days ago
9-33639
9 days
33990 YaelDillies
author:YaelDillies
chore(SetTheory/Cardinal): remove explicit argument to `nat_lt_aleph0` It is almost never used. Also rename to `natCast_lt_aleph0` and add `natCast_le_aleph0`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-set-theory 88/100 Mathlib/Algebra/Lie/CartanExists.lean,Mathlib/Algebra/Module/LinearMap/Polynomial.lean,Mathlib/FieldTheory/CardinalEmb.lean,Mathlib/FieldTheory/Cardinality.lean,Mathlib/FieldTheory/Finite/Polynomial.lean,Mathlib/FieldTheory/Fixed.lean,Mathlib/FieldTheory/SeparableClosure.lean,Mathlib/GroupTheory/CoprodI.lean,Mathlib/LinearAlgebra/Dimension/Constructions.lean,Mathlib/LinearAlgebra/Dimension/ErdosKaplansky.lean,Mathlib/LinearAlgebra/Dimension/Finite.lean,Mathlib/LinearAlgebra/Dimension/Finrank.lean,Mathlib/LinearAlgebra/Dimension/StrongRankCondition.lean,Mathlib/ModelTheory/Encoding.lean,Mathlib/Order/Filter/Cocardinal.lean,Mathlib/RingTheory/AlgebraicIndependent/TranscendenceBasis.lean,Mathlib/RingTheory/MvPolynomial/Homogeneous.lean,Mathlib/SetTheory/Cardinal/Aleph.lean,Mathlib/SetTheory/Cardinal/Arithmetic.lean,Mathlib/SetTheory/Cardinal/Basic.lean,Mathlib/SetTheory/Cardinal/Continuum.lean,Mathlib/SetTheory/Cardinal/Divisibility.lean,Mathlib/SetTheory/Cardinal/ENat.lean,Mathlib/SetTheory/Cardinal/Finite.lean,Mathlib/SetTheory/Cardinal/Free.lean,Mathlib/SetTheory/Cardinal/Ordinal.lean,Mathlib/SetTheory/Cardinal/Regular.lean,Mathlib/SetTheory/Cardinal/ToNat.lean,Mathlib/SetTheory/Ordinal/Basic.lean,Mathlib/Topology/MetricSpace/GromovHausdorff.lean 30 3 ['YaelDillies', 'github-actions', 'vihdzp'] nobody
0-2041
34 minutes ago
unknown
unknown
32882 DavidLedvinka
author:DavidLedvinka
feat(Probability): add `Adapted ` Add `Adapted` which is a version of `StronglyAdapted` for `Measurable `rather than `StronglyMeasurable`. Also add theorems which state when one property implies the other and when they are equivalent. - [x] depends on: #33063 t-measure-probability delegated 65/95 Mathlib/Probability/Kernel/Disintegration/Density.lean,Mathlib/Probability/Martingale/BorelCantelli.lean,Mathlib/Probability/Martingale/Centering.lean,Mathlib/Probability/Martingale/Upcrossing.lean,Mathlib/Probability/Process/Adapted.lean,Mathlib/Probability/Process/Stopping.lean 6 8 ['DavidLedvinka', 'RemyDegenne', 'github-actions', 'kex-y', 'mathlib-bors', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] kex-y
assignee:kex-y
0-1909
31 minutes ago
0-1909
28 minutes ago
3-24094
3 days
33790 eliasjudin
author:eliasjudin
feat(CategoryTheory/Preadditive/Mat): add natural transformation and isomorphism extension theorems --- - Add `Mat_.natTrans_ext`, an extensionality lemma showing that a natural transformation `F ⟶ G` between functors `Mat_ C ⥤ D` (with `G` additive) is determined by its components on objects of the form `(embedding C).obj X`. - Add `Mat_.liftIso_ext_comp_embeddingLiftIso`, a small uniqueness lemma for comparisons `L ≅ lift F`. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory new-contributor awaiting-author 42/3 Mathlib/CategoryTheory/Preadditive/Mat.lean 1 12 ['eliasjudin', 'github-actions', 'joelriou', 'kim-em'] nobody
0-1859
30 minutes ago
5-51706
5 days ago
0-20054
5 hours
33991 grunweg
author:grunweg
test: pretty-printing of class abbrev Lake build fails with an error in batteries: what am I doing wrong? --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) file-removed large-import 118/303 .github/workflows/daily.yml,Mathlib.lean,Mathlib/Algebra/Group/Action/TransferInstance.lean,Mathlib/Algebra/Group/TypeTags/Basic.lean,Mathlib/Algebra/Notation/Defs.lean,Mathlib/Algebra/Notation/Lemmas.lean,Mathlib/Algebra/Notation/Pi/Defs.lean,Mathlib/Algebra/Notation/Prod.lean,Mathlib/Algebra/Order/Group/Defs.lean,Mathlib/Algebra/Order/Group/Unbundled/Basic.lean,Mathlib/CategoryTheory/Limits/Yoneda.lean,Mathlib/Data/Finite/Defs.lean,Mathlib/Data/Int/Cast/Pi.lean,Mathlib/Data/Int/Init.lean,Mathlib/Data/List/Flatten.lean,Mathlib/Data/List/GetD.lean,Mathlib/Data/List/Indexes.lean,Mathlib/Data/Multiset/Defs.lean,Mathlib/Data/Nat/Basic.lean,Mathlib/Data/Nat/Bits.lean,Mathlib/Data/Nat/Init.lean,Mathlib/GroupTheory/GroupAction/SubMulAction/OfFixingSubgroup.lean,Mathlib/Lean/Meta/Simp.lean,Mathlib/Order/BoundedOrder/Basic.lean,Mathlib/Order/GaloisConnection/Defs.lean,Mathlib/Order/Monotone/Defs.lean,Mathlib/RingTheory/Valuation/Discrete/Basic.lean,Mathlib/SetTheory/Cardinal/Defs.lean,Mathlib/Tactic/Common.lean,Mathlib/Tactic/FunProp/Decl.lean,Mathlib/Tactic/Linter/DirectoryDependency.lean,Mathlib/Tactic/NormNum/Core.lean,Mathlib/Tactic/Positivity/Core.lean,Mathlib/Tactic/Push/Attr.lean,Mathlib/Tactic/Widget/LibraryRewrite.lean,Mathlib/Topology/Defs/Basic.lean,Mathlib/Util/AssertExists.lean,MathlibTest/AssertExists.lean,MathlibTest/CalcQuestionMark.lean,MathlibTest/DeprecatedSyntaxLinter.lean,MathlibTest/DirectoryDependencyLinter/Test.lean,MathlibTest/EmptyLine.lean,MathlibTest/ExtractGoal.lean,MathlibTest/HaveLetLinter.lean,MathlibTest/LibrarySearch/IsCompact.lean,MathlibTest/LintStyle.lean,MathlibTest/TacticAnalysis.lean,MathlibTest/UnusedInstancesInType.lean,MathlibTest/Util/PrintSorries.lean,MathlibTest/WhitespaceLinter.lean,MathlibTest/aesop_cat.lean,MathlibTest/eqns.lean,MathlibTest/fast_instance.lean,MathlibTest/globalAttributeIn.lean,MathlibTest/hintAll.lean,MathlibTest/jacobiSym.lean,MathlibTest/slim_check.lean,MathlibTest/toAdditive.lean,lake-manifest.json,lakefile.lean,lean-toolchain 61 1 ['github-actions'] nobody
0-1737
28 minutes ago
unknown
unknown
33896 loefflerd
author:loefflerd
refactor(Geometry/Manifold): split long file ChartedSpace.lean Split the > 1500 line file `Mathlib.Geometry.Manifold.ChartedSpace` into 3 shorter files. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-differential-geometry tech debt ready-to-merge 935/868 Mathlib.lean,Mathlib/Geometry/Manifold/ChartedSpace.lean,Mathlib/Geometry/Manifold/ConformalGroupoid.lean,Mathlib/Geometry/Manifold/HasGroupoid.lean,Mathlib/Geometry/Manifold/IsManifold/Basic.lean,Mathlib/Geometry/Manifold/LocalInvariantProperties.lean,Mathlib/Geometry/Manifold/StructureGroupoid.lean 7 2 ['github-actions', 'jcommelin'] grunweg
assignee:grunweg
0-1636
27 minutes ago
0-1636
24 minutes ago
2-30387
2 days
33915 tb65536
author:tb65536
feat: irreducible components of schemes --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP t-ring-theory t-algebra t-algebraic-geometry large-import awaiting-author
label:t-algebra$
655/140 Mathlib/Algebra/Module/LocalizedModule/Submodule.lean,Mathlib/AlgebraicGeometry/IrreducibleComponents.lean,Mathlib/RingTheory/Ideal/Colon.lean,Mathlib/RingTheory/Ideal/IsPrimary.lean,Mathlib/RingTheory/IsPrimary.lean,Mathlib/RingTheory/Lasker.lean 6 4 ['erdOne', 'github-actions', 'tb65536'] nobody
0-1540
25 minutes ago
unknown
unknown
30122 xroblot
author:xroblot
Development branch (1) --- WIP large-import 4127/23 Mathlib.GaloisTower.lean,Mathlib/AddCharTrace.lean,Mathlib/Algebra/Group/Subgroup/Basic.lean,Mathlib/Algebra/Group/Subgroup/Map.lean,Mathlib/Algebra/Group/Submonoid/BigOperators.lean,Mathlib/Algebra/Group/Submonoid/Operations.lean,Mathlib/Algebra/Group/Submonoid/Units.lean,Mathlib/Algebra/MvPolynomial/Eval.lean,Mathlib/Cyclotomic.lean,Mathlib/Data/Nat/Digits/Lemmas.lean,Mathlib/Duality.lean,Mathlib/FieldTheory/IntermediateField/Adjoin/Basic.lean,Mathlib/FieldTheory/PrimeField.lean,Mathlib/GalCyclotomic.lean,Mathlib/GaussSum.lean,Mathlib/GroupTheory/Exponent.lean,Mathlib/GroupTheory/FiniteAbelian/Duality.lean,Mathlib/GroupTheory/QuotientGroup/Basic.lean,Mathlib/KroneckerWeber_Blueprint.lean,Mathlib/Logic/Equiv/Set.lean,Mathlib/MWE.lean,Mathlib/Misc.lean,Mathlib/NumberTheory/MulChar/Basic.lean,Mathlib/NumberTheory/MulChar/Duality.lean,Mathlib/NumberTheory/MulChar/Lemmas.lean,Mathlib/NumberTheory/NumberField/Ideal/KummerDedekind.lean,Mathlib/RingTheory/Ideal/Int.lean,Mathlib/RingTheory/Ideal/Over.lean,Mathlib/RingTheory/Ideal/Pointwise.lean,Mathlib/RingTheory/RootsOfUnity/Basic.lean,Mathlib/StickElt.lean,Mathlib/Teichmuller.lean 32 10 ['github-actions', 'mathlib4-merge-conflict-bot'] nobody
0-1341
22 minutes ago
unknown
unknown
33988 leanprover-community-bot-assistant
author:leanprover-community-bot-assistant
chore: remove declarations deprecated between 2021-01-15 and 2025-07-15 I am happy to remove some deprecated declarations for you! Please check if there are any remaining stray comments or other issues before merging. --- [workflow run for this PR](https://github.com/leanprover-community/mathlib4/actions/runs/21019723123) 0/976 Mathlib/Algebra/Algebra/Shrink.lean,Mathlib/Algebra/Category/ModuleCat/Monoidal/Basic.lean,Mathlib/Algebra/Group/Pointwise/Finset/Basic.lean,Mathlib/Algebra/GroupWithZero/Range.lean,Mathlib/Algebra/Module/Shrink.lean,Mathlib/Algebra/Module/Submodule/Map.lean,Mathlib/Algebra/Polynomial/FieldDivision.lean,Mathlib/Analysis/Convex/Cone/InnerDual.lean,Mathlib/Analysis/InnerProductSpace/Adjoint.lean,Mathlib/Analysis/InnerProductSpace/GramSchmidtOrtho.lean,Mathlib/Analysis/InnerProductSpace/Projection/Basic.lean,Mathlib/Analysis/InnerProductSpace/Projection/Submodule.lean,Mathlib/CategoryTheory/Dialectica/Monoidal.lean,Mathlib/CategoryTheory/GradedObject/Monoidal.lean,Mathlib/CategoryTheory/Localization/Monoidal/Basic.lean,Mathlib/CategoryTheory/Monoidal/Braided/Basic.lean,Mathlib/CategoryTheory/Monoidal/Cartesian/Basic.lean,Mathlib/CategoryTheory/Noetherian.lean,Mathlib/Combinatorics/Additive/Energy.lean,Mathlib/Data/Fin/Tuple/Basic.lean,Mathlib/Data/Rel.lean,Mathlib/Data/Set/Card.lean,Mathlib/Geometry/Manifold/VectorBundle/Tangent.lean,Mathlib/Geometry/Manifold/VectorField/LieBracket.lean,Mathlib/GroupTheory/DoubleCoset.lean,Mathlib/GroupTheory/FreeAbelianGroup.lean,Mathlib/GroupTheory/GroupAction/SubMulAction/OfStabilizer.lean,Mathlib/LinearAlgebra/CrossProduct.lean,Mathlib/LinearAlgebra/Lagrange.lean,Mathlib/LinearAlgebra/Projection.lean,Mathlib/LinearAlgebra/RootSystem/Defs.lean,Mathlib/LinearAlgebra/RootSystem/Reduced.lean,Mathlib/LinearAlgebra/Span/Defs.lean,Mathlib/LinearAlgebra/TensorProduct/Basic.lean,Mathlib/MeasureTheory/Integral/Lebesgue/Basic.lean,Mathlib/NumberTheory/NumberField/InfinitePlace/Ramification.lean,Mathlib/NumberTheory/PrimeCounting.lean,Mathlib/NumberTheory/SmoothNumbers.lean,Mathlib/Order/Atoms.lean,Mathlib/Order/CompleteLattice/Basic.lean,Mathlib/Order/Concept.lean,Mathlib/Order/Filter/Basic.lean,Mathlib/Order/IsNormal.lean,Mathlib/Order/RelSeries.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/Functoriality.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/LongExactSequence.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/LowDegree.lean,Mathlib/RingTheory/FiniteType.lean,Mathlib/RingTheory/Ideal/Pointwise.lean,Mathlib/RingTheory/Polynomial/ContentIdeal.lean,Mathlib/SetTheory/Cardinal/Aleph.lean,Mathlib/SetTheory/Cardinal/Regular.lean,Mathlib/SetTheory/Game/Nim.lean,Mathlib/SetTheory/Ordinal/Arithmetic.lean,Mathlib/SetTheory/Ordinal/Exponential.lean,Mathlib/SetTheory/Ordinal/Family.lean,Mathlib/SetTheory/Ordinal/Principal.lean,Mathlib/SetTheory/Ordinal/Topology.lean,Mathlib/Topology/AlexandrovDiscrete.lean,Mathlib/Topology/Compactness/NhdsKer.lean,Mathlib/Topology/ContinuousOn.lean,Mathlib/Topology/Defs/Filter.lean,Mathlib/Topology/NhdsKer.lean,Mathlib/Topology/OmegaCompletePartialOrder.lean,Mathlib/Topology/Order/LawsonTopology.lean,Mathlib/Topology/Order/ScottTopology.lean 66 7 ['Ruben-VandeVelde', 'github-actions'] nobody
0-939
15 minutes ago
unknown
unknown
33643 vihdzp
author:vihdzp
feat: `r < stdPart x → r < x` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) ready-to-merge t-algebra
label:t-algebra$
30/19 Mathlib/Algebra/Order/Ring/StandardPart.lean 1 7 ['YaelDillies', 'github-actions', 'jcommelin', 'vihdzp'] dagurtomas
assignee:dagurtomas
0-776
12 minutes ago
0-778
9 minutes ago
8-76247
8 days
33390 farmanb
author:farmanb
feat(RingTheory/Ideal): generalize Submodule.colon to sets This PR generalizes `Submodule.colon` to arguments of type `Set M` in the second slot and updates the surrounding API accordingly. Main changes * Generalize `Submodule.colon` to take `S : Set M` rather than `P : Submodule R M`. * Normalize theorems/lemmas to use `Set.univ` instead of `⊤` where appropriate. * Strengthen `iInf_colon_iSup` by removing an unnecessary commutativity assumption. * Update monotonicity and inclusion lemmas (e.g. `_root_.Ideal.le_colon`) to use set inclusions. * Add `colon_bot'` (`CommSemiring`): identify `⊥.colon S` with the annihilator of `Submodule.span R S`. * Adjust annihilator-related proofs to account for the generalized colon, using explicit coercions such as `Submodule.top_coe`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-ring-theory new-contributor 113/54 Mathlib/RingTheory/Ideal/Colon.lean,Mathlib/RingTheory/Ideal/Oka.lean,Mathlib/RingTheory/Lasker.lean,Mathlib/RingTheory/Noetherian/OfPrime.lean,Mathlib/RingTheory/PrincipalIdealDomainOfPrime.lean,Mathlib/RingTheory/Support.lean 6 67 ['erdOne', 'farmanb', 'github-actions', 'tb65536'] nobody
0-737
12 minutes ago
0-20533
5 hours ago
4-59904
4 days
33920 Citronhat
author:Citronhat
feat(topology): generalize tendsto_inv_iff from ℝ≥0∞ to topological groups This PR implements the [TODO](https://github.com/leanprover-community/mathlib4/blob/b2f24e70b375e42e5a60251a2f43baa20ca668f1/Mathlib/Topology/Instances/ENNReal/Lemmas.lean#L468C1-L471C70) in `Topology.Instances.ENNReal.Lemmas` by moving the lemma to a more general setting. - Add a general lemma `tendsto_inv_iff` in `Topology.Algebra.Group.Basic` (with `@[simp]`), whose proof is the same as the previous `ℝ≥0∞` proof, just stated for an arbitrary `G` with `[InvolutiveInv G]` and `[ContinuousInv G]`. - Mark it `@[to_additive (attr := simp)]`, so the additive analogue is generated automatically. - Change `ENNReal.tendsto_inv_iff` in `Topology.Instances.ENNReal.Lemmas` to be a wrapper around the new lemma, preserving the existing statement/attributes and avoiding duplication. No mathematical content changes: this is a relocation/generalization of the existing proof plus the additive version. t-topology new-contributor 11/9 Mathlib/MeasureTheory/Covering/Differentiation.lean,Mathlib/MeasureTheory/Integral/Lebesgue/Markov.lean,Mathlib/Topology/Algebra/Group/Basic.lean,Mathlib/Topology/Instances/ENNReal/Lemmas.lean 4 4 ['Citronhat', 'github-actions', 'vihdzp'] nobody
0-497
8 minutes ago
0-3876
1 hour ago
1-35816
1 day
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). --- - [x] depends on: #31205 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis t-convex-geometry ready-to-merge 62/0 Mathlib/Analysis/Convex/Side.lean 1 4 ['YaelDillies', 'github-actions', 'jcommelin', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] YaelDillies
assignee:YaelDillies
0-477
7 minutes ago
0-478
4 minutes ago
37-85221
37 days

Other lists of PRs

Some other lists of PRs which could be useful:

PRs with non-conforming titles

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
25474 adomani
author:adomani
test for .lean/.md check A test PR for #25473. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-linter file-removed 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
163-84340
5 months ago
unknown
unknown
29605 alreadydone
author:alreadydone
experiment(Algebra): unbundle npow/zpow from Monoid/InvDivMonoid --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict t-algebra awaiting-CI
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
121-61826
3 months ago
unknown
unknown
30421 grunweg
author:grunweg
WIP: support products in the differential geometry elaborators Nothing to see yet. Best reviewed commit by commit. --- - [ ] depends on: #30413 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
78-83931
2 months ago
96-40240
96 days ago
0-1188
19 minutes
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author t-algebra new-contributor
label:t-algebra$
47/0 Mathlib/Algebra/Group/Subgroup/Pointwise.lean 1 10 ['FrederickPu', 'eric-wieser', 'github-actions', 'plp127', 'tb65536'] nobody
78-69838
2 months ago
87-59872
87 days ago
0-40723
11 hours
30121 idontgetoutmuch
author:idontgetoutmuch
Principal fiber bundle core A structure capturing what it means to be a principal fibre bundle. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author t-differential-geometry new-contributor 227/0 Mathlib.lean,Mathlib/Geometry/Manifold/PrincipalFiberBundle/PrincipalGBundle.lean 2 6 ['github-actions', 'grunweg', 'mathlib4-merge-conflict-bot'] hrmacbeth
assignee:hrmacbeth
57-5479
1 month ago
79-65335
79 days ago
24-28967
24 days
31102 JOSHCLUNE
author:JOSHCLUNE
Require LeanHammer Experimenting with adding LeanHammer as a mathlib dependency --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict new-contributor 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
57-4969
1 month ago
unknown
unknown
31339 grunweg
author:grunweg
Movelemma --- - [ ] depends on: #31338 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
56-68117
1 month ago
69-30833
69 days ago
0-1120
18 minutes
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/361 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 18 ['eric-wieser', 'github-actions', 'kim-em', 'mathlib4-merge-conflict-bot'] nobody
37-13827
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory large-import merge-conflict 133/46 Mathlib/CategoryTheory/Bicategory/InducedBicategory.lean,Mathlib/CategoryTheory/Category/Grpd.lean,Mathlib/CategoryTheory/ConcreteCategory/Bundled.lean 3 6 ['Jlh18', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
28-46933
28 days ago
unknown
unknown
33707 jcommelin
author:jcommelin
ci: add commit verification for transient and automated commits This PR adds a CI workflow that verifies PRs correctly use transient and automated commits, and provides reviewers with a clear summary of which commits need human review. Commit types: - **Substantive commits**: Regular commits requiring human review - **Automated commits** (`x: `): CI verifies the commit is the exact result of running the command on the parent - **Transient commits** (`transient: ...`): CI verifies these have zero net effect on the final tree What this PR adds: - `scripts/verify_commits.sh` - Main verification script - `scripts/verify_commits_summary.sh` - Generates PR comment from JSON output - `.github/workflows/commit_verification.yml` - GitHub Actions workflow --- ### Testing locally The commit at `HEAD^` contains test branch creation scripts. These can be used for testing the functionality of the two shell scripts. To test: ```bash # Checkout the commit with test scripts git checkout HEAD^ # Create a test branch based on your current branch (before checkout) # Save your branch name first: BASE_BRANCH=$(git rev-parse --abbrev-ref HEAD) git checkout HEAD^ ./scripts/create_test_branch.sh $BASE_BRANCH # Run verification (should pass) ./scripts/verify_commits.sh $BASE_BRANCH ./scripts/verify_commits.sh $BASE_BRANCH --json | ./scripts/verify_commits_summary.sh repo_foo 12345 # Clean up and return git checkout $BASE_BRANCH && git branch -D ci-x-test-* ``` Available test scripts: - `create_test_branch.sh` - Creates a branch with valid transient + auto commits (should pass) - `create_test_branch_fail_conflict.sh` - Transient commits cause cherry-pick conflicts (should fail) - `create_test_branch_fail_transient.sh` - Transient commits have net effect (should fail) - `create_test_branch_fail_auto.sh` - Auto commit doesn't match command output (should fail) 🤖 Generated with [Claude Code](https://claude.com/claude-code) CI merge-conflict 685/0 .github/workflows/commit_verification.yml,scripts/verify_commits.sh,scripts/verify_commits_summary.sh 3 2 ['github-actions', 'mathlib4-merge-conflict-bot'] nobody
7-27849
7 days ago
7-27850
7 days ago
0-55642
15 hours
33714 idontgetoutmuch
author:idontgetoutmuch
Riemannian metrics exist II Supersedes https://github.com/leanprover-community/mathlib4/pull/33519 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-differential-geometry new-contributor 1269/0 Mathlib.lean,Mathlib/Geometry/Manifold/ExistsRiemannianMetricTangentSpace.lean,Mathlib/Geometry/Manifold/PartitionOfUnity.lean 3 3 ['github-actions', 'grunweg', 'idontgetoutmuch'] PatrickMassot
assignee:PatrickMassot
3-31254
3 days ago
6-85595
6 days ago
6-85415
6 days
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author CI merge-conflict 1/1 bors.toml 1 5 ['bryangingechen', 'eric-wieser', 'github-actions', 'mathlib4-merge-conflict-bot', 'urkud'] nobody
3-19388
3 days ago
75-55184
75 days ago
0-64037
17 hours
33743 jcommelin
author:jcommelin
ci: add automated commit verification This PR adds verification for "x: " commits that checks whether re-running the command produces the same tree. Written with the help of Claude Code. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) CI 406/28 .github/workflows/commit_verification.yml,scripts/README.md,scripts/verify_commits.sh,scripts/verify_commits_summary.sh 4 6 ['Vierkantor', 'github-actions', 'jcommelin'] joneugster
assignee:joneugster
2-31263
2 days ago
7-3255
7 days ago
7-3075
7 days
33044 bryangingechen
author:bryangingechen
ci: also get cache for parent commit cf. https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Mathlib.20has.20moved.20to.20the.20new.20module.20system/near/563452000 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) CI 84/8 .github/build.in.yml,.github/workflows/bors.yml,.github/workflows/build.yml,.github/workflows/build_fork.yml 4 7 ['bryangingechen', 'github-actions', 'jcommelin', 'mathlib-bors'] joneugster
assignee:joneugster
0-70882
19 hours ago
0-70951
19 hours ago
26-31071
26 days
33979 adomani
author:adomani
ci: add `splice-bot` action Adds a CI action that inspects review comments. If a review comment selects at least one line and contains the string `splice-bot` at the start of some line, then the bot will create a PR with just the changes to the selected file, clearing all history. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) CI 16/0 .github/workflows/splice_bot.yaml 1 2 ['bryangingechen', 'github-actions'] bryangingechen
assignee:bryangingechen
0-41314
11 hours ago
unknown
unknown
33991 grunweg
author:grunweg
test: pretty-printing of class abbrev Lake build fails with an error in batteries: what am I doing wrong? --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) file-removed large-import 118/303 .github/workflows/daily.yml,Mathlib.lean,Mathlib/Algebra/Group/Action/TransferInstance.lean,Mathlib/Algebra/Group/TypeTags/Basic.lean,Mathlib/Algebra/Notation/Defs.lean,Mathlib/Algebra/Notation/Lemmas.lean,Mathlib/Algebra/Notation/Pi/Defs.lean,Mathlib/Algebra/Notation/Prod.lean,Mathlib/Algebra/Order/Group/Defs.lean,Mathlib/Algebra/Order/Group/Unbundled/Basic.lean,Mathlib/CategoryTheory/Limits/Yoneda.lean,Mathlib/Data/Finite/Defs.lean,Mathlib/Data/Int/Cast/Pi.lean,Mathlib/Data/Int/Init.lean,Mathlib/Data/List/Flatten.lean,Mathlib/Data/List/GetD.lean,Mathlib/Data/List/Indexes.lean,Mathlib/Data/Multiset/Defs.lean,Mathlib/Data/Nat/Basic.lean,Mathlib/Data/Nat/Bits.lean,Mathlib/Data/Nat/Init.lean,Mathlib/GroupTheory/GroupAction/SubMulAction/OfFixingSubgroup.lean,Mathlib/Lean/Meta/Simp.lean,Mathlib/Order/BoundedOrder/Basic.lean,Mathlib/Order/GaloisConnection/Defs.lean,Mathlib/Order/Monotone/Defs.lean,Mathlib/RingTheory/Valuation/Discrete/Basic.lean,Mathlib/SetTheory/Cardinal/Defs.lean,Mathlib/Tactic/Common.lean,Mathlib/Tactic/FunProp/Decl.lean,Mathlib/Tactic/Linter/DirectoryDependency.lean,Mathlib/Tactic/NormNum/Core.lean,Mathlib/Tactic/Positivity/Core.lean,Mathlib/Tactic/Push/Attr.lean,Mathlib/Tactic/Widget/LibraryRewrite.lean,Mathlib/Topology/Defs/Basic.lean,Mathlib/Util/AssertExists.lean,MathlibTest/AssertExists.lean,MathlibTest/CalcQuestionMark.lean,MathlibTest/DeprecatedSyntaxLinter.lean,MathlibTest/DirectoryDependencyLinter/Test.lean,MathlibTest/EmptyLine.lean,MathlibTest/ExtractGoal.lean,MathlibTest/HaveLetLinter.lean,MathlibTest/LibrarySearch/IsCompact.lean,MathlibTest/LintStyle.lean,MathlibTest/TacticAnalysis.lean,MathlibTest/UnusedInstancesInType.lean,MathlibTest/Util/PrintSorries.lean,MathlibTest/WhitespaceLinter.lean,MathlibTest/aesop_cat.lean,MathlibTest/eqns.lean,MathlibTest/fast_instance.lean,MathlibTest/globalAttributeIn.lean,MathlibTest/hintAll.lean,MathlibTest/jacobiSym.lean,MathlibTest/slim_check.lean,MathlibTest/toAdditive.lean,lake-manifest.json,lakefile.lean,lean-toolchain 61 1 ['github-actions'] nobody
0-1737
28 minutes ago
unknown
unknown

PRs without an area label

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
24100 eric-wieser
author:eric-wieser
feat: restore some explicit binders from Lean 3 Part of #24099 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author tech debt 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
234-70461
7 months ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
98-85635
3 months ago
98-85636
98 days ago
25-73895
25 days
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] --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR new-contributor 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
96-64841
3 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict file-removed 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
72-63099
2 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR large-import new-contributor 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
63-23317
2 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR large-import new-contributor 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
63-23316
2 months ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
59-48551
1 month ago
unknown
unknown
29411 llllvvuu
author:llllvvuu
feat(LinearAlgebra/Matrix/Rank): rank factorization The rank factorization derived from `Module.finBasis`. Co-authored-by: Aristotle Harmonic --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
57-6120
1 month ago
82-71897
82 days ago
46-47927
46 days
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
57-5320
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
57-5314
1 month ago
97-58071
97 days ago
0-2352
39 minutes
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR large-import 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
56-64885
1 month ago
unknown
unknown
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. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
50-17088
1 month ago
68-79400
68 days ago
9-65641
9 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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
47-59879
1 month 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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author merge-conflict 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
44-35474
1 month ago
51-84726
51 days ago
6-67021
6 days
29000 JovanGerb
author:JovanGerb
feat(Tactic/Push): add basic tags and tests This PR adds basic `@[push]` tags, and expands the `push` test file. --- - [ ] depends on: #21965 - [ ] depends on: #30038 - [ ] depends on: #30039 - [ ] depends on: #30042 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
40-51531
1 month ago
109-28139
109 days ago
0-9867
2 hours
32609 PrParadoxy
author:PrParadoxy
feat(LinearAlgebra/PiTensorProduct): Relation between nested tensor products and tensor products indexed by dependent sums Product tensors in `⨂ j : (Σ i, β i), s j.fst j.snd` can be mapped to product tensors in `⨂ i, ⨂ b : β i, s i b`. If the outer index type is finite, the two types are equivalent. This allows the definition of endomorphisms on PiTensorProducts by specifying them on disjoint subsets of the index set. Such constructions are common e.g. in quantum circuits, quantum cellular automata, and renormalization procedures. --- WIP. This PR contains two "requests for comments". Essentially: * Is a single complex-to-define linear equivalence preferable over several less complex ones, which might however be of limited interest by themselves? * Which trade-offs are appropriate to make things computable? - [ ] depends on: #32608 - [ ] depends on: #32600 - [x] depends on: #32598 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor blocked-by-other-PR 683/0 Mathlib.lean,Mathlib/Data/Sigma/Basic.lean,Mathlib/LinearAlgebra/Multilinear/Basic.lean,Mathlib/LinearAlgebra/PiTensorProduct/Nested.lean,Mathlib/LinearAlgebra/PiTensorProduct/Set.lean 5 4 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
34-32413
1 month ago
37-43788
37 days ago
0-614
10 minutes
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 merge-conflict 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 5 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
34-12623
1 month ago
84-11942
84 days ago
0-1475
24 minutes
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
33-67964
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
33-67963
1 month ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](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
33-67960
1 month ago
unknown
unknown
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 - [x] depends on: #30236 - [x] depends on: #30202 - [x] depends on: #30201 - [x] depends on: #30199 - [x] depends on: #30198 - [x] depends on: #30197 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR merge-conflict 463/18 Mathlib/Analysis/Distribution/ContDiffMapSupportedIn.lean 1 5 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
33-67959
1 month ago
unknown
unknown
32600 PrParadoxy
author:PrParadoxy
feat(LinearAlgebra/Multilinear): composition of multilinear maps The composition of a multilinear map with a family of multilinear maps is a multilinear map indexed by a dependent sum. The result reduces to a lemma about the interaction of function application, `Sigma.curry`, and `Function.update`. This variant of `Function.apply_update` is included as `Sigma.apply_curry_update`. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor 40/0 Mathlib/Data/Sigma/Basic.lean,Mathlib/LinearAlgebra/Multilinear/Basic.lean 2 4 ['github-actions', 'goliath-klein', 'kbuzzard'] dwrensha
assignee:dwrensha
31-60260
1 month ago
unknown
unknown
32829 Hagb
author:Hagb
feat(Data/Finsupp/MonomialOrder): weaken `IsOrderedCancelAddMonoid` to `IsOrderedAddMonoid` `IsOrderedCancelAddMonoid syn` (`.iocam`) can be obtained from `IsOrderedAddMonoid syn` and other fields. --- - [ ] depends on: #32828 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR 11/2 Mathlib/Algebra/Order/Group/Defs.lean,Mathlib/Data/Finsupp/MonomialOrder.lean 2 5 ['Hagb', 'github-actions', 'mathlib4-dependent-issues-bot', 'vihdzp'] nobody
30-63702
30 days ago
unknown
unknown
33016 xgenereux
author:xgenereux
feat: RingHom.adjoinAlgebraMap Consider a tower of rings `A / B / C` and `b : B`, then there is a natural map from `A[b]` to `A[algebraMap B C b]` (adjoin `b` viewed as an element of `C`). This PR adds 3 versions, depending on whether we use `Algebra.adjoin` or `IntermediateField.adjoin`: - `Algebra.RingHom.adjoinAlgebraMap : Algebra.adjoin A {b} →+* Algebra.adjoin A {(algebraMap B C) b}` - `IntermediateField.RingHom.adjoinAlgebraMapOfAlgebra : Algebra.adjoin A {b} →+* A⟮((algebraMap B C) b)⟯` - `IntermediateField.RingHom.adjoinAlgebraMap : A⟮b⟯ →+* A⟮((algebraMap B C) b)⟯` Note: We create a new file for `Algebra.RingHom.adjoinAlgebraMap`, which is intended for results about adjoining singletons, because it is convenient to import `Algebra.Adjoin.Polynomial`. Co-authored-by: María Inés de Frutos Fernández <[mariaines.dff@gmail.com](mailto:mariaines.dff@gmail.com)> --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 103/0 Mathlib.lean,Mathlib/FieldTheory/IntermediateField/Adjoin/Algebra.lean,Mathlib/FieldTheory/IntermediateField/Adjoin/Defs.lean,Mathlib/RingTheory/Adjoin/Singleton.lean 4 1 ['github-actions'] bryangingechen
assignee:bryangingechen
25-31238
25 days ago
28-37014
28 days ago
28-36834
28 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 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] --> [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author new-contributor large-import 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
25-29725
25 days ago
115-84846
115 days ago
2-2914
2 days
32983 JovanGerb
author:JovanGerb
feat: use `LE.le` for subset relation in `Set`, `Finset`, `PSet`, `ZFSet` This PR allows the use of `⊆` notation while the underlying constant is `≤`. Similarly for `⊂`/`<`, `⊇`/`≥` and `⊃`/`>`. Hmm, seemingly still a lot of build failures --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict 248/159 Mathlib/Algebra/Group/Pointwise/Set/Basic.lean,Mathlib/Algebra/MonoidAlgebra/Support.lean,Mathlib/Combinatorics/Matroid/Basic.lean,Mathlib/Combinatorics/SetFamily/AhlswedeZhang.lean,Mathlib/Data/Finset/Defs.lean,Mathlib/Data/Finset/Filter.lean,Mathlib/Data/Finset/Image.lean,Mathlib/Data/Finset/Lattice/Basic.lean,Mathlib/Data/Fintype/Card.lean,Mathlib/Data/Multiset/ZeroCons.lean,Mathlib/Data/Rat/Star.lean,Mathlib/Data/Set/Basic.lean,Mathlib/Data/Set/Defs.lean,Mathlib/Data/Set/FiniteExhaustion.lean,Mathlib/Data/Set/Sups.lean,Mathlib/Data/SetLike/Basic.lean,Mathlib/Data/SetNotation.lean,Mathlib/MeasureTheory/SetSemiring.lean,Mathlib/Order/Birkhoff.lean,Mathlib/Order/BooleanAlgebra/Basic.lean,Mathlib/Order/Booleanisation.lean,Mathlib/Order/Bounds/Basic.lean,Mathlib/Order/CountableDenseLinearOrder.lean,Mathlib/Order/Filter/Basic.lean,Mathlib/Order/Heyting/Basic.lean,Mathlib/Order/RelClasses.lean,Mathlib/Order/SupIndep.lean,Mathlib/RingTheory/WittVector/StructurePolynomial.lean,Mathlib/SetTheory/ZFC/Basic.lean,Mathlib/SetTheory/ZFC/Class.lean,Mathlib/SetTheory/ZFC/PSet.lean,Mathlib/Topology/Compactness/SigmaCompact.lean,Mathlib/Topology/UniformSpace/Basic.lean 33 2 ['github-actions', 'mathlib4-merge-conflict-bot'] nobody
24-58455
24 days ago
unknown
unknown
33109 felixpernegger
author:felixpernegger
feat(Data/Nat/Choose): Binomial inversion This PR adds binomial inversion (also called binomial transform), which is a useful method for proving binomial identities. It is tricky to find direct references to binomial inversion, but for example [this](https://en.wikipedia.org/wiki/Binomial_transform#Binomial_convolution) Wikipedia article mentions it ("The formula"). The first theorem ```alternating_sum_choose_mul_of_alternating_sum_choose_mul``` could be refined (we only need the hypothesis ```h``` up to some point), but this seems to needlessly complicate it. new-contributor 107/0 Mathlib.lean,Mathlib/Data/Nat/Choose/Inversion.lean 2 4 ['felixpernegger', 'github-actions', 'wwylele'] dagurtomas
assignee:dagurtomas
23-31251
23 days ago
25-62272
25 days ago
26-4033
26 days
32987 kim-em
author:kim-em
feat: pipeline downloads and decompression in `cache get` This PR modifies `lake exe cache get` to decompress files as they download, rather than waiting for all downloads to complete first. Previously the cache system had two sequential phases: download all files using `curl --parallel`, then decompress all files using a single `leantar` call. Now a background task spawns sequential batched `leantar` calls to decompress files as downloads complete, pipelining network I/O and disk I/O. 🤖 Prepared with Claude Code 194/30 Cache/Requests.lean 1 1 ['github-actions'] dagurtomas
assignee:dagurtomas
18-31230
18 days ago
28-32215
28 days ago
29-29019
29 days
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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR large-import 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
17-34139
17 days ago
unknown
unknown
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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import 227/2 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
17-33856
17 days ago
17-31509
17 days ago
64-13257
64 days
33143 wwylele
author:wwylele
feat(PowerSeries): pentagonal number theorem The proof is split in two files: `Mathlib/Topology/Algebra/InfiniteSum/Pentagonal.lean` for the algebraic part, and `Mathlib/RingTheory/PowerSeries/Pentagonal.lean` for the summability part. In the near future, I also plan to prove the real/complex version that branches off from the algebraic part. --- - [ ] depends on: #30436 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 324/1 Mathlib.lean,Mathlib/RingTheory/PowerSeries/Pentagonal.lean,Mathlib/Topology/Algebra/InfiniteSum/Pentagonal.lean,docs/1000.yaml 4 12 ['copilot-pull-request-reviewer', 'github-actions', 'mathlib4-dependent-issues-bot', 'vihdzp'] kex-y
assignee:kex-y
16-31261
16 days ago
18-69044
18 days ago
19-38681
19 days
33406 dupuisf
author:dupuisf
feat: add basics of majorization This PR defines [majorization](https://en.wikipedia.org/wiki/Majorization). This is needed to develop the theory of unitarily invariant norms on `ℂ^n`, in particular Schatten norms. --- - [ ] depends on: #33394 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR 784/15 Mathlib.lean,Mathlib/Analysis/Convex/DoublyStochasticMatrix.lean,Mathlib/Analysis/Convex/Majorization/Basic.lean,Mathlib/Analysis/Convex/Majorization/Defs.lean,Mathlib/Data/Finset/BooleanAlgebra.lean,Mathlib/Data/Finset/Card.lean,Mathlib/Data/Finset/Image.lean,Mathlib/Data/Finset/Max.lean,Mathlib/Data/Finset/Powerset.lean,Mathlib/Data/Fintype/Card.lean,Mathlib/Order/Interval/Finset/Fin.lean 11 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
15-19472
15 days ago
unknown
unknown
33276 NicolaBernini
author:NicolaBernini
feat: Rename List.reverse_perm to List.reverse_perm_self and List.reverse_perm' to List.reverse_perm_iff --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor awaiting-author 17/15 Mathlib/Algebra/BigOperators/Group/List/Basic.lean,Mathlib/Data/Finset/Dedup.lean,Mathlib/Data/List/Basic.lean,Mathlib/Data/List/Defs.lean,Mathlib/Data/List/Perm/Lattice.lean,Mathlib/Data/List/Permutation.lean,Mathlib/Data/Multiset/Defs.lean,Mathlib/NumberTheory/Divisors.lean 8 4 ['Ruben-VandeVelde', 'github-actions'] kim-em
assignee:kim-em
12-68503
12 days ago
16-78697
16 days ago
3-79472
3 days
33463 khwilson
author:khwilson
feat(Mathlib/Analysis/Polynomial/MahlerMeasure): Mahler Measure for other rings Define `mahlerMeasure'` which allows you specify a norm preserving map `v` from any `NormedRing A` (or more general) to `ℂ`. Also provide wrappers around the main `mahlerMeasure` lemmas that are used for estimation. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor 96/2 Mathlib/Analysis/Polynomial/MahlerMeasure.lean,Mathlib/NumberTheory/MahlerMeasure.lean 2 16 ['github-actions', 'khwilson', 'plp127', 'vlad902'] nobody
11-64316
11 days ago
unknown
unknown
32608 PrParadoxy
author:PrParadoxy
feat(LinearAlgebra/PiTensorProduct): API for PiTensorProducts indexed by sets This PR addresses a TODO item in LinearAlgebra/PiTensorProduct.lean: * API for the various ways ι can be split into subsets; connect this with the binary tensor product -- specifically by describing tensors of type ⨂ (i : S), M i, for S : Set ι. Our primary motivation is to formalise the notion of "restricted tensor products". This will be the content of a follow-up PR. Beyond that, the Set API is natural in contexts where the index type has an independent interpretation. An example is quantum physics, where ι ranges over distinguishable degrees of freedom, and where its is common practice to annotate objects by the set of indices they are defined on. --- Stub file with preliminary definition of the restricted tensor product as a direct limit of tensors indexed by finite subsets of an index type: https://github.com/PrParadoxy/mathlib4/blob/restricted-stub/Mathlib/LinearAlgebra/PiTensorProduct/Restricted.lean --- - [x] depends on: #32598 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor awaiting-zulip 300/2 Mathlib.lean,Mathlib/LinearAlgebra/PiTensorProduct.lean,Mathlib/LinearAlgebra/PiTensorProduct/Set.lean 3 28 ['PrParadoxy', 'dagurtomas', 'eric-wieser', 'github-actions', 'goliath-klein', 'leanprover-radar', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] dagurtomas
assignee:dagurtomas
11-59342
11 days ago
23-59045
23 days ago
10-63624
10 days
30927 callesonne
author:callesonne
feat(Bicategory/Yoneda): add the yoneda pseudofunctor --- - [ ] depends on: #30926 - [x] depends on: #30895 - [x] depends on: #25901 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 81/3 Mathlib.lean,Mathlib/CategoryTheory/Bicategory/Basic.lean,Mathlib/CategoryTheory/Bicategory/Yoneda.lean,Mathlib/CategoryTheory/Category/Cat.lean,Mathlib/Data/Opposite.lean 5 4 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
10-77542
10 days ago
unknown
unknown
33469 erdOne
author:erdOne
feat(LinearAlgebra): make TensorProduct.finsuppLeft and friends heterobasic --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 77/137 Mathlib/LinearAlgebra/DirectSum/Finsupp.lean,Mathlib/LinearAlgebra/DirectSum/TensorProduct.lean,Mathlib/LinearAlgebra/TensorProduct/Basis.lean,Mathlib/LinearAlgebra/TensorProduct/Submodule.lean,Mathlib/RepresentationTheory/Coinvariants.lean,Mathlib/RepresentationTheory/Rep.lean,Mathlib/RingTheory/Flat/FaithfullyFlat/Basic.lean,Mathlib/RingTheory/Ideal/Quotient/Index.lean,Mathlib/RingTheory/LocalRing/Module.lean,Mathlib/RingTheory/Localization/BaseChange.lean,Mathlib/RingTheory/PicardGroup.lean,Mathlib/RingTheory/TensorProduct/IsBaseChangeFree.lean,Mathlib/RingTheory/TensorProduct/MvPolynomial.lean 13 1 ['github-actions'] mariainesdff
assignee:mariainesdff
10-31233
10 days ago
13-33944
13 days ago
13-33764
13 days
33470 erdOne
author:erdOne
feat: generalize `Polynomial.freeMonic` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 80/52 Mathlib.lean,Mathlib/Algebra/Polynomial/FreeMonic.lean,Mathlib/RingTheory/Polynomial/UniversalFactorizationRing.lean 3 1 ['github-actions'] thorimur
assignee:thorimur
10-31233
10 days ago
13-39501
13 days ago
13-39321
13 days
32585 CBirkbeck
author:CBirkbeck
feat(NumberTheory/ModularForms/EisensteinSeries/E2/Transform): E2 under the action of SL2 We show how E2 transforms under the slash action of SL2. --- - [x] depends on : #32584 - [x] depends on : #32955 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 466/0 Mathlib.lean,Mathlib/NumberTheory/ModularForms/EisensteinSeries/E2/Summable.lean,Mathlib/NumberTheory/ModularForms/EisensteinSeries/E2/Transform.lean 3 11 ['CBirkbeck', 'github-actions', 'loefflerd', 'mathlib4-merge-conflict-bot'] loefflerd
assignee:loefflerd
9-56315
9 days ago
9-56315
9 days ago
12-53590
12 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 - [x] depends on: #29230 for `Lattice` `CompleteLattice` - [ ] depends on: #29241 for the definition of `orthogonal` blocked-by-other-PR 243/6 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
9-43980
9 days ago
134-72213
134 days ago
0-1521
25 minutes
33281 michelsol
author:michelsol
feat(Analysis/SpecialFunctions/Integrals): integral of 1/sqrt(1-x^2) and its integrability. Add the integral of the derivative of arcsin and its integrability. --- - [ ] depends on: #33280 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor blocked-by-other-PR merge-conflict 59/0 Mathlib/Analysis/SpecialFunctions/Integrability/Basic.lean,Mathlib/Analysis/SpecialFunctions/Integrals/Basic.lean,Mathlib/MeasureTheory/Integral/IntervalIntegral/FundThmCalculus.lean 3 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
9-35221
9 days ago
20-54035
20 days ago
0-811
13 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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR large-import 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
9-10681
9 days ago
unknown
unknown
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. --- - [x] depends on: #31998 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 243/0 Mathlib.lean,Mathlib/RingTheory/LocalProperties/ProjectiveDimension.lean 2 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
9-3082
9 days ago
9-11219
9 days ago
13-18336
13 days
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR 1108/10 Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Baer.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/Algebra/Homology/DerivedCategory/Ext/Map.lean,Mathlib/Algebra/Homology/DerivedCategory/ShortExact.lean,Mathlib/Algebra/Homology/HomotopyCategory/Pretriangulated.lean,Mathlib/Algebra/Homology/HomotopyCategory/ShortExact.lean,Mathlib/Algebra/Homology/ShortComplex/ModuleCat.lean,Mathlib/Algebra/Order/Monoid/Unbundled/WithTop.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/RingTheory/Noetherian/Basic.lean,Mathlib/RingTheory/Regular/InjectiveDimension.lean 15 4 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
8-74751
8 days ago
50-71451
50 days ago
0-294
4 minutes
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR 1099/0 Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Baer.lean,Mathlib/Algebra/Category/ModuleCat/Ext/DimensionShifting.lean,Mathlib/Algebra/Category/ModuleCat/Ext/Ulift.lean,Mathlib/Algebra/Category/ModuleCat/InjectiveDimension.lean,Mathlib/Algebra/Category/ModuleCat/Ulift.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/Bijection.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/EnoughInjectives.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/EnoughProjectives.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/Map.lean,Mathlib/Algebra/Homology/DerivedCategory/ShortExact.lean,Mathlib/Algebra/Homology/HomotopyCategory/Pretriangulated.lean,Mathlib/Algebra/Homology/HomotopyCategory/ShortExact.lean,Mathlib/Algebra/Homology/ShortComplex/ModuleCat.lean,Mathlib/RingTheory/Gorenstein/Defs.lean,Mathlib/RingTheory/Noetherian/Basic.lean 16 4 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
8-74388
8 days ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR 450/0 Mathlib.lean,Mathlib/RingTheory/LocalProperties/Injective.lean,Mathlib/RingTheory/LocalProperties/InjectiveDimension.lean 3 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
8-74230
8 days ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR 1651/0 Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Baer.lean,Mathlib/Algebra/Category/ModuleCat/Ext/DimensionShifting.lean,Mathlib/Algebra/Category/ModuleCat/Ext/Ulift.lean,Mathlib/Algebra/Category/ModuleCat/InjectiveDimension.lean,Mathlib/Algebra/Category/ModuleCat/Ulift.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/Bijection.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/EnoughInjectives.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/EnoughProjectives.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/Map.lean,Mathlib/Algebra/Homology/DerivedCategory/ShortExact.lean,Mathlib/Algebra/Homology/HomotopyCategory/Pretriangulated.lean,Mathlib/Algebra/Homology/HomotopyCategory/ShortExact.lean,Mathlib/Algebra/Homology/ShortComplex/ModuleCat.lean,Mathlib/RingTheory/Gorenstein/Basic.lean,Mathlib/RingTheory/Gorenstein/Defs.lean,Mathlib/RingTheory/LocalProperties/Injective.lean,Mathlib/RingTheory/LocalProperties/InjectiveDimension.lean,Mathlib/RingTheory/Noetherian/Basic.lean 19 5 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
8-74159
8 days ago
unknown
unknown
33369 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`. --- - [ ] depends on: #31046 - [ ] depends on: #31222 - [ ] depends on: #32316 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import blocked-by-other-PR 948/0 Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Ext/BaseChange.lean,Mathlib/Algebra/Category/ModuleCat/Ext/DimensionShifting.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/EnoughInjectives.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/EnoughProjectives.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/Map.lean,Mathlib/Algebra/Homology/DerivedCategory/ShortExact.lean,Mathlib/Algebra/Homology/HomotopyCategory/Pretriangulated.lean,Mathlib/Algebra/Homology/HomotopyCategory/ShortExact.lean,Mathlib/Algebra/Homology/ShortComplex/ModuleCat.lean,Mathlib/Algebra/Module/FinitePresentation.lean,Mathlib/RingTheory/Flat/IsBaseChange.lean,Mathlib/RingTheory/Noetherian/Basic.lean 13 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
8-72081
8 days ago
16-77822
16 days ago
0-535
8 minutes
33377 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: #33369 - [ ] depends on: #31884 - [ ] depends on: #32098 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import blocked-by-other-PR 2590/10 Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Baer.lean,Mathlib/Algebra/Category/ModuleCat/Ext/BaseChange.lean,Mathlib/Algebra/Category/ModuleCat/Ext/DimensionShifting.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/Ext/Bijection.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/EnoughInjectives.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/EnoughProjectives.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/Map.lean,Mathlib/Algebra/Homology/DerivedCategory/ShortExact.lean,Mathlib/Algebra/Homology/HomotopyCategory/Pretriangulated.lean,Mathlib/Algebra/Homology/HomotopyCategory/ShortExact.lean,Mathlib/Algebra/Homology/ShortComplex/ModuleCat.lean,Mathlib/Algebra/Module/FinitePresentation.lean,Mathlib/Algebra/Order/Monoid/Unbundled/WithTop.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/RingTheory/Flat/IsBaseChange.lean,Mathlib/RingTheory/Gorenstein/Defs.lean,Mathlib/RingTheory/Gorenstein/Polynomial.lean,Mathlib/RingTheory/Noetherian/Basic.lean,Mathlib/RingTheory/Regular/InjectiveDimension.lean 24 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
8-71895
8 days ago
unknown
unknown
33379 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: #31884 - [ ] depends on: #26218 - [ ] depends on: #32098 - [ ] depends on: #31644 - [ ] depends on: #33369 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import blocked-by-other-PR 5059/26 Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Baer.lean,Mathlib/Algebra/Category/ModuleCat/Ext/BaseChange.lean,Mathlib/Algebra/Category/ModuleCat/Ext/DimensionShifting.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/Ext/Bijection.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/EnoughInjectives.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/EnoughProjectives.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/Map.lean,Mathlib/Algebra/Homology/DerivedCategory/ShortExact.lean,Mathlib/Algebra/Homology/HomotopyCategory/Pretriangulated.lean,Mathlib/Algebra/Homology/HomotopyCategory/ShortExact.lean,Mathlib/Algebra/Homology/ShortComplex/ModuleCat.lean,Mathlib/Algebra/Module/FinitePresentation.lean,Mathlib/Algebra/Order/Monoid/Unbundled/WithTop.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/Noetherian/Basic.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 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
8-71760
8 days ago
unknown
unknown
33380 Thmoas-Guan
author:Thmoas-Guan
feat(RingTheory): Gorenstein local ring is Cohen--Macaulay local ring of type one 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: #33379 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import blocked-by-other-PR 6010/26 Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Baer.lean,Mathlib/Algebra/Category/ModuleCat/Ext/BaseChange.lean,Mathlib/Algebra/Category/ModuleCat/Ext/DimensionShifting.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/Ext/Bijection.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/EnoughInjectives.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/EnoughProjectives.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/Map.lean,Mathlib/Algebra/Homology/DerivedCategory/ShortExact.lean,Mathlib/Algebra/Homology/HomotopyCategory/Pretriangulated.lean,Mathlib/Algebra/Homology/HomotopyCategory/ShortExact.lean,Mathlib/Algebra/Homology/ShortComplex/ModuleCat.lean,Mathlib/Algebra/Module/FinitePresentation.lean,Mathlib/Algebra/Order/Monoid/Unbundled/WithTop.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/Noetherian/Basic.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 31 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
8-71653
8 days 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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR large-import 2627/30 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/Algebra/Homology/ShortComplex/ModuleCat.lean,Mathlib/Algebra/Order/Monoid/Unbundled/WithTop.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/RingTheory/CohenMacaulay/Basic.lean,Mathlib/RingTheory/CohenMacaulay/Maximal.lean,Mathlib/RingTheory/Ideal/Cotangent.lean,Mathlib/RingTheory/KrullDimension/Regular.lean,Mathlib/RingTheory/Noetherian/Basic.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 18 8 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
8-70448
8 days ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR large-import 3125/30 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/Algebra/Homology/ShortComplex/ModuleCat.lean,Mathlib/Algebra/Order/Monoid/Unbundled/WithTop.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/RingTheory/CohenMacaulay/Basic.lean,Mathlib/RingTheory/CohenMacaulay/Maximal.lean,Mathlib/RingTheory/Ideal/Cotangent.lean,Mathlib/RingTheory/KrullDimension/Regular.lean,Mathlib/RingTheory/Noetherian/Basic.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 20 8 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
8-70381
8 days ago
unknown
unknown
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author blocked-by-other-PR 683/0 Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Baer.lean,Mathlib/Algebra/Category/ModuleCat/Ext/DimensionShifting.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/EnoughInjectives.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/EnoughProjectives.lean,Mathlib/Algebra/Homology/ShortComplex/ModuleCat.lean,Mathlib/RingTheory/GlobalDimension.lean,Mathlib/RingTheory/LocalProperties/ProjectiveDimension.lean,Mathlib/RingTheory/Noetherian/Basic.lean 9 13 ['Thmoas-Guan', 'github-actions', 'jcommelin', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
8-69386
8 days ago
51-994
51 days ago
1-66277
1 day
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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR large-import 3432/30 Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Baer.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/Algebra/Homology/ShortComplex/ModuleCat.lean,Mathlib/Algebra/Order/Monoid/Unbundled/WithTop.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/RingTheory/CohenMacaulay/Basic.lean,Mathlib/RingTheory/CohenMacaulay/Maximal.lean,Mathlib/RingTheory/GlobalDimension.lean,Mathlib/RingTheory/Ideal/Cotangent.lean,Mathlib/RingTheory/KrullDimension/Regular.lean,Mathlib/RingTheory/Noetherian/Basic.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 22 11 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
8-69321
8 days 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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR large-import 3831/30 Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Baer.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/Algebra/Homology/ShortComplex/ModuleCat.lean,Mathlib/Algebra/Order/Monoid/Unbundled/WithTop.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/RingTheory/CohenMacaulay/Basic.lean,Mathlib/RingTheory/CohenMacaulay/Maximal.lean,Mathlib/RingTheory/GlobalDimension.lean,Mathlib/RingTheory/Ideal/Cotangent.lean,Mathlib/RingTheory/KrullDimension/Regular.lean,Mathlib/RingTheory/LocalProperties/ProjectiveDimension.lean,Mathlib/RingTheory/Noetherian/Basic.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 25 12 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
8-69308
8 days 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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR large-import 2938/30 Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Baer.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/Algebra/Homology/ShortComplex/ModuleCat.lean,Mathlib/Algebra/Order/Monoid/Unbundled/WithTop.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/RingTheory/GlobalDimension.lean,Mathlib/RingTheory/Ideal/Cotangent.lean,Mathlib/RingTheory/KrullDimension/Regular.lean,Mathlib/RingTheory/Noetherian/Basic.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 20 9 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
8-69262
8 days 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 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR large-import 4630/30 Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Baer.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/Algebra/Homology/ShortComplex/ModuleCat.lean,Mathlib/Algebra/Order/Monoid/Unbundled/WithTop.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/RingTheory/CohenMacaulay/Basic.lean,Mathlib/RingTheory/CohenMacaulay/Maximal.lean,Mathlib/RingTheory/GlobalDimension.lean,Mathlib/RingTheory/Ideal/Cotangent.lean,Mathlib/RingTheory/KrullDimension/Regular.lean,Mathlib/RingTheory/LocalProperties/ProjectiveDimension.lean,Mathlib/RingTheory/Noetherian/Basic.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 28 12 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
8-69231
8 days ago
unknown
unknown
32742 LTolDe
author:LTolDe
feat(MeasureTheory/Constructions/Polish/Basic): add class SuslinSpace add new class `SuslinSpace` for a topological space that is an analytic set in itself This will be useful to prove the **Effros Theorem**, see [zulip thread](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Effros.20Theorem/with/558712441). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor awaiting-zulip 4/0 Mathlib/MeasureTheory/Constructions/Polish/Basic.lean 1 9 ['ADedecker', 'LTolDe', 'dupuisf', 'github-actions', 'jcommelin'] PatrickMassot
assignee:PatrickMassot
8-65927
8 days ago
8-66080
8 days ago
11-6345
11 days
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 `#min_imports` does not give a correct set of imports. - [x] 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` blocked-by-other-PR 601/7 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
8-62947
8 days ago
unknown
unknown
33314 YuvalFilmus
author:YuvalFilmus
feat(Trigonometric/Chebyshev/Basic): calculate iterated derivatives of T and U at 1 Added theorems for the iterated derivatives of T and U at 1. These formulas are fractions, and so I also added theorems stating that the denominator divides the numerator. --- - [ ] depends on: #33312 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR 148/0 Mathlib/Analysis/SpecialFunctions/Trigonometric/Chebyshev/Basic.lean,Mathlib/RingTheory/Polynomial/Chebyshev.lean 2 4 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
6-84264
6 days ago
19-60764
19 days ago
0-882
14 minutes
33275 YuvalFilmus
author:YuvalFilmus
feat(Trigonometric/Chebyshev/Extremal): Chebyshev polynomials maximize iterated derivatives We prove that Chebyshev polynomials maximized iterated derivatives at points x≥1. --- - [ ] depends on: #33259 - [ ] depends on: #33274 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR 423/22 Mathlib.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Chebyshev/Extremal.lean,Mathlib/Data/Finset/Powerset.lean,Mathlib/LinearAlgebra/Lagrange.lean 4 4 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
6-59617
6 days ago
unknown
unknown
33274 YuvalFilmus
author:YuvalFilmus
feat(LinearAlgebra/Lagrange): Formula for iterated derivative of a polynomial using Lagrange interpolation We give a formula for the iterated derivative of a polynomial at a point using Lagrange interpolation. This will be used to prove that Chebyshev polynomials maximize iterated derivatives at points x≥1. --- - [x] depends on: #33161 - [x] depends on: #33193 - [ ] depends on: #33194 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR 106/22 Mathlib/Data/Finset/Powerset.lean,Mathlib/LinearAlgebra/Lagrange.lean 2 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
6-57542
6 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 408/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
6-30318
6 days ago
unknown
unknown
33555 erdOne
author:erdOne
feat(RingTheory): standard smooth = etale over mvpolynomial --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import 79/2 Mathlib/Algebra/MvPolynomial/Equiv.lean,Mathlib/Algebra/MvPolynomial/PDeriv.lean,Mathlib/RingTheory/RingHom/StandardSmooth.lean 3 3 ['erdOne', 'github-actions', 'robin-carlier'] robin-carlier
assignee:robin-carlier
5-81803
5 days ago
10-50529
10 days ago
10-50349
10 days
33594 smmercuri
author:smmercuri
feat: `HeightOneSpectrum.valuation` is rank one for number fields - If `K` is a number field and `v` is a height-one prime ideal then `v.valuation K` is rank one. - In general, if `v` is a rank one valuation of `K`, then its extension to the `v`-adic completion `v.Completion` is also rank one, provided in `Valuation.instRankOneCompletion` - Together these refactor and deprecate `instRankOneValuedAdicCompletion`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import 18/8 Mathlib/NumberTheory/NumberField/FinitePlaces.lean,Mathlib/RingTheory/Valuation/RankOne.lean 2 2 ['github-actions', 'smmercuri'] jcommelin
assignee:jcommelin
5-31261
5 days ago
9-73677
9 days ago
9-73497
9 days
33662 Pjotr5
author:Pjotr5
feat(Algebra/Order/BigOperators/Expect): add lemmas and strict variants ### Summary - Combine `le_expect_nonempty_of_subadditive` and `le_expect_of_subadditive` into a single lemma `le_expect_of_subadditive`. The extra assumptions `(hs : s.Nonempty)` and `(h_zero : m 0 = 0)` are unnecessary (since `m 0 = 0` follows from `h_div`). This requires a small downstream update to `Mathlib/Analysis/RCLike/Basic.lean` (`norm_expect_le`). - Add strict-inequality variants: `expect_lt_expect`, `expect_lt`, `lt_expect`. - Add existence lemmas: `exists_le_of_expect_le_expect`, `exists_le_of_le_expect`, `exists_le_of_expect_le`, and `exists_lt_of_expect_lt_expect`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor 46/16 Mathlib/Algebra/Order/BigOperators/Expect.lean,Mathlib/Analysis/RCLike/Basic.lean 2 1 ['github-actions'] dagurtomas
assignee:dagurtomas
5-31257
5 days ago
8-83692
8 days ago
8-84432
8 days
31795 thorimur
author:thorimur
feat: turn on `unusedFintypeInType` linter This PR turns on the `unusedFintypeInType` linter introduced in #31794 by adding it to the `mathlibStandardSet` of linters in Mathlib.Init. --- - [ ] depends on: #31794 - [x] depends on: #33068 - [x] depends on: #33148 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR merge-conflict file-removed 311/46 Mathlib/Data/Fintype/EquivFin.lean,Mathlib/Data/Fintype/Quotient.lean,Mathlib/Init.lean,Mathlib/Tactic/Linter/UnusedInstancesInType.lean,MathlibTest/UnusedInstancesInType/Basic.lean,MathlibTest/UnusedInstancesInType/Decidable.lean,MathlibTest/UnusedInstancesInType/Fintype.lean,MathlibTest/UnusedInstancesInType/FintypeNeedingImport.lean,MathlibTest/UnusedInstancesInType/SetOption.lean 9 10 ['SnirBroshi', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'thorimur'] nobody
4-53876
4 days ago
unknown
unknown
33312 YuvalFilmus
author:YuvalFilmus
feat(Polynomial/Chebyshev): formulas for iterated derivatives of T and U at 1 The main results are `iterate_derivative_T_eval_one` and `iterate_derivative_U_eval_one`. These are derived using recurrences which for at every point, and in particular, `iterate_derivative_T_eval_zero` and `iterate_derivative_U_eval_zero` gives the recurrences at zero. In principle, by combining with #33311, one can compute the explicit formula for the derivative at zero. A subsequent PR will derive consequences for these polynomials over the reals (these should work for every field). The file is getting rather long — not sure what to do about it. --- - [ ] depends on: #33283 - [ ] depends on: #33306 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 110/0 Mathlib/RingTheory/Polynomial/Chebyshev.lean 1 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] Vierkantor
assignee:Vierkantor
3-31256
3 days ago
7-51576
7 days ago
7-52899
7 days
33791 PhoenixIra
author:PhoenixIra
feat: Generalization of FixedPointApproximants to CompletePartialOrder --- This PR provides a generalization of FixedPointApproximants to CompletePartialOrder. Not every theorem can be generalized, as sometimes we require additional conditions (namely `x ≤ f x`) in order to guarantee that the set is directed and thus the supremum is well-defined. This is not necessary in a CompleteLattice. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor 255/42 Mathlib/Order/CompletePartialOrder.lean,Mathlib/SetTheory/Ordinal/FixedPointApproximants.lean 2 7 ['github-actions', 'vihdzp'] vihdzp
assignee:vihdzp
3-29241
3 days ago
unknown
unknown
33863 urkud
author:urkud
feat: generalize some lemmas about LTOs Currently, lemmas about `Filter.map ((↑) : Set.Iio a → X) Filter.atTop` etc assume that the ambient type is densely ordered. However, it suffices to require that `a` is an `Order.IsSuccPrelimit`. Make this generalization and move the lemmas to a new file. Also, use the new lemmas to drop a `[DenselyOrdered _]` assumption in one lemma in measure theory. These more precise statements are also useful when dealing with, e.g., LTOs defined by ordinals. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 226/130 Mathlib.lean,Mathlib/Analysis/SpecialFunctions/Exp.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Arctan.lean,Mathlib/MeasureTheory/Measure/Hausdorff.lean,Mathlib/MeasureTheory/Measure/MeasureSpace.lean,Mathlib/Topology/Order/AtTopBotIxx.lean,Mathlib/Topology/Order/DenselyOrdered.lean 7 1 ['github-actions'] nobody
3-17890
3 days ago
3-16171
3 days ago
3-15991
3 days
33864 Timeroot
author:Timeroot
feat(Computability/Primrec): Proving several Nat arithmetic functions are primrec Prove that gcd, lcm, coprimality, divisiblity, primality, factorial, descending factorial, powers, and various logarithms are all primitive recursive. Co-authored-by: Aristotle Harmonic <[aristotle-harmonic@harmonic.fun](mailto:aristotle-harmonic@harmonic.fun)> large-import 195/4 Mathlib.lean,Mathlib/Computability/Primrec.lean,Mathlib/Computability/Primrec/List.lean,Mathlib/Computability/Primrec/Nat.lean,Mathlib/Data/Nat/Log.lean 5 5 ['eric-wieser', 'github-actions', 'mathlib4-merge-conflict-bot'] nobody
2-44024
2 days ago
2-26141
2 days ago
2-25961
2 days
33736 fbarroero
author:fbarroero
feat(RingTheory/Polynomial/GaussNorm): The `gaussNorm` is an absolute value if `v` is a nonarchimedean absolute value We prove ``` Polynomial.gaussNorm_isAbsoluteValue {c : ℝ} {R : Type*} [Ring R] {v : AbsoluteValue R ℝ} (hna : IsNonarchimedean v) (hc : 0 < c) : IsAbsoluteValue (gaussNorm v c) ``` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 194/7 Mathlib/Algebra/Order/AbsoluteValue/Basic.lean,Mathlib/Algebra/Order/Ring/IsNonarchimedean.lean,Mathlib/RingTheory/Polynomial/GaussNorm.lean 3 4 ['copilot-pull-request-reviewer', 'github-actions'] ADedecker
assignee:ADedecker
2-31264
2 days ago
5-60767
5 days ago
5-60587
5 days
33757 fpvandoorn
author:fpvandoorn
feat: remove decidability instances on sets or ideals * We have the rule that you should assume decidability instead of opening the classical locale. However, in places where there cannot ever be a reasonable decidable instance, I think we can relax this rule. * This PR updates the corresponding library note, and removes `DecidableEq` instances on `Set` and `Ideal` * This looks a lot cleaner IMO, and the decidability assumptions are silly: assuming that `Set α` has decidable for an inhabited type `α` is equivalent to assuming that all propositions are decidable. Similarly for `Ideal R` for a nontrivial ring `R`. * This has one downside: if a lemma uses classical logic to infer decidability for its statement, then all lemmas that use this lemma also have to do this, otherwise they will deal with decidability type mismatches --- This was motivated by seeing some code from @mariainesdff's repos with such decidability arguments. @mariainesdff, do you think this PR would make your code a bit nicer? [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 57/32 Mathlib/Algebra/Module/DedekindDomain.lean,Mathlib/Algebra/Module/PID.lean,Mathlib/Logic/Basic.lean,Mathlib/MeasureTheory/SetSemiring.lean,Mathlib/NumberTheory/RamificationInertia/Basic.lean,Mathlib/Order/PartialSups.lean,Mathlib/RingTheory/DedekindDomain/Factorization.lean,Mathlib/RingTheory/DedekindDomain/Ideal/Lemmas.lean,Mathlib/RingTheory/Ideal/Basic.lean,Mathlib/RingTheory/Invariant/Basic.lean,Mathlib/RingTheory/Lasker.lean,Mathlib/RingTheory/Valuation/ValuationRing.lean 12 5 ['github-actions', 'plp127', 'vihdzp'] nobody
2-5221
2 days ago
6-61042
6 days ago
6-60862
6 days
32757 AntoineChambert-Loir
author:AntoineChambert-Loir
feat(LinearAlgebra/Transvection): the determinant of a transvection is equal to 1. Prove 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$$. --- - [x] depends on: #31138 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 255/0 Mathlib/LinearAlgebra/Determinant.lean,Mathlib/LinearAlgebra/Transvection.lean 2 10 ['AntoineChambert-Loir', 'alreadydone', 'eric-wieser', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
1-69817
1 day ago
1-64763
1 day ago
23-10004
23 days
33634 xgenereux
author:xgenereux
feat(ValuationSubring): eq_self_or_eq_top_of_le Using `primeSpectrumEquiv` we get the the corresponding results of `IsLocalRing.primeSpectrum_eq_of_KrullDimLEOne`(see #33607) for valuation subrings. --- - [ ] depends on: #33631 - [ ] depends on: #33612 - [ ] depends on: #33609 - [ ] depends on: #33607 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR large-import 79/18 Mathlib/Algebra/Order/Ring/Ordering/Basic.lean,Mathlib/RingTheory/DedekindDomain/Ideal/Lemmas.lean,Mathlib/RingTheory/Ideal/GoingUp.lean,Mathlib/RingTheory/Ideal/Maps.lean,Mathlib/RingTheory/Ideal/Maximal.lean,Mathlib/RingTheory/Ideal/MinimalPrime/Basic.lean,Mathlib/RingTheory/Ideal/NatInt.lean,Mathlib/RingTheory/Ideal/Prime.lean,Mathlib/RingTheory/Jacobson/Ring.lean,Mathlib/RingTheory/KrullDimension/Basic.lean,Mathlib/RingTheory/KrullDimension/Zero.lean,Mathlib/RingTheory/LocalRing/ResidueField/Fiber.lean,Mathlib/RingTheory/Localization/Ideal.lean,Mathlib/RingTheory/Spectrum/Prime/Basic.lean,Mathlib/RingTheory/Spectrum/Prime/Topology.lean,Mathlib/RingTheory/Valuation/ValuationSubring.lean 16 6 ['alreadydone', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'plp127', 'xgenereux'] nobody
1-43977
1 day ago
unknown
unknown
33882 AntoineChambert-Loir
author:AntoineChambert-Loir
feat(LinearAlgebra/Transvection/SpecialLinearGroup): commutators in the special linear group Over a field, prove the following results : * transvections are conjugate in the general linear group; except in rank 2, they are conjugate in the special linear group. * the special linear group is equal to its commutator subgroup (except when it doesn't, ie, in rank 2 over a field with 2 or 3 elements). --- - [ ] depends on: #33347 - [ ] depends on: #33348 - [ ] depends on: #33387 - [ ] depends on: #33282 - [ ] depends on: #33392 - [ ] depends on: #33402 - [ ] depends on: #33485 - [ ] depends on: #32757 - [ ] depends on: #33560 - [ ] depends on: #33692 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR file-removed 3128/235 Mathlib.lean,Mathlib/GroupTheory/Commutator/Basic.lean,Mathlib/LinearAlgebra/Basis/Fin.lean,Mathlib/LinearAlgebra/Center.lean,Mathlib/LinearAlgebra/Determinant.lean,Mathlib/LinearAlgebra/Dual/Defs.lean,Mathlib/LinearAlgebra/FiniteDimensional/Lemmas.lean,Mathlib/LinearAlgebra/LinearIndependent/Lemmas.lean,Mathlib/LinearAlgebra/SpecialLinearGroup.lean,Mathlib/LinearAlgebra/Transvection.lean,Mathlib/LinearAlgebra/Transvection/Basic.lean,Mathlib/LinearAlgebra/Transvection/Generation.lean,Mathlib/LinearAlgebra/Transvection/SpecialLinearGroup.lean 13 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
1-40634
1 day ago
unknown
unknown
33631 xgenereux
author:xgenereux
feat(ValuationSubring): simp lemmas for idealOfLE/ofPrime in relation to top/bot simp lemmas for `idealOfLE`/`ofPrime` in the trivial cases of `⊥`, `⊤` . This is my second try at this PR (after I bailed on #33618), sorry about this! --- - [ ] depends on: #33612 - [ ] depends on: #33609 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR 30/0 Mathlib/RingTheory/Valuation/ValuationSubring.lean 1 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
1-38886
1 day ago
unknown
unknown
33964 JovanGerb
author:JovanGerb
feat(Order/Interval/Set): `to_dual` for `Iio`/`Iic` This PR tags `Iio`/`Ioi` and `Iic`/`Ici` with `to_dual`. Unfortuately we can't do this yet for `Ioc`/`Ico` and `Ioo` and `Icc`, as we need to have #32438 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 101/219 Mathlib/Order/Interval/Set/Basic.lean,Mathlib/Order/Interval/Set/Defs.lean,Mathlib/Tactic/Translate/ToDual.lean 3 2 ['JovanGerb', 'github-actions'] nobody
0-62993
17 hours ago
unknown
unknown
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. The violations found by this linter are fixed in #33068 (merged) and #33148 (merged). Note that the portion of this diff corresponding to the actual linter file is relatively small (+68 -11), and is very similar to the `unusedDecidableInType` linter. The majority of the diff in the linter file itself is factoring out the workaround to lean4#11313 (which is used in both linters); the rest of the diff comes from reorganizing tests and adding tests. --- - [x] depends on: #31142 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) maintainer-merge file-removed 304/46 Mathlib/Tactic/Linter/UnusedInstancesInType.lean,MathlibTest/UnusedInstancesInType/Basic.lean,MathlibTest/UnusedInstancesInType/Decidable.lean,MathlibTest/UnusedInstancesInType/Fintype.lean,MathlibTest/UnusedInstancesInType/FintypeNeedingImport.lean,MathlibTest/UnusedInstancesInType/SetOption.lean 6 15 ['JovanGerb', 'github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'thorimur'] JovanGerb
assignee:JovanGerb
0-62542
17 hours ago
2-48797
2 days ago
40-21713
40 days
29942 smmercuri
author:smmercuri
feat(InfinitePlace/Completion): embeddings of `w.Completion` factor through embeddings of `v.Completion` when `w` extends `v` If `w : InfinitePlace L` and `v : InfinitePlace K` to `L` are such that we have `Algebra v.Completion w.Completion`, then `extensionEmbedding w : L →+* ℂ` factors through `extensionEmbedding v : K →+* ℂ` (provided the algebras are well behaved). --- - [x] depends on: #27978 - [x] depends on: #29969 - [x] depends on: #29944 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) FLT 102/15 Mathlib/Analysis/Normed/Field/WithAbs.lean,Mathlib/NumberTheory/NumberField/InfinitePlace/Completion.lean,Mathlib/NumberTheory/NumberField/InfinitePlace/Embeddings.lean,Mathlib/Topology/MetricSpace/Completion.lean 4 6 ['github-actions', 'joelriou', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] nobody
0-49364
13 hours ago
0-48456
13 hours ago
47-37031
47 days
33834 JovanGerb
author:JovanGerb
feat(CategoryTheory/NatTrans): use to_dual This PR tags `NatTrans` with `to_dual`. The two functor arguments get swapped because the underlying `NatTrans.app` has its direction swapped. Translating the `naturality` field is slightly awkward. We need to define a constant `naturality'` (analogously to `Category.assoc') --- - [ ] depends on: #33237 - [ ] depends on: #33777 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 11/3 Mathlib/CategoryTheory/NatTrans.lean 1 3 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
0-43044
11 hours ago
0-40651
11 hours ago
0-40471
11 hours
33916 AntoineChambert-Loir
author:AntoineChambert-Loir
feat(LinearAlgebra/SpecialLinearGroup/Simple): simplicity of the projective special linear group. Let `K` be a field and `V` be a `K`-vector space. * `SpecialLinearGroup.isQuasiSimpleGroup`: if `finrank K V` is at least 3, or if `finrank K V = 2` and `K` has at least 4 elements, then `SpecialLinearGroup K V` is quasi-simple, namely, the quotient group `SpecialLinearGroup K V ⧸ Subgroup.center (SpecialLinearGroup K V)` is simple. --- - [ ] depends on: #33347 - [ ] depends on: #33348 - [ ] depends on: #33387 - [ ] depends on: #33282 - [ ] depends on: #33392 - [ ] depends on: #33402 - [ ] depends on: #33485 - [ ] depends on: #32757 - [ ] depends on: #33560 - [ ] depends on: #33692 - [ ] depends on: #33882 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) file-removed large-import blocked-by-other-PR 3527/239 Mathlib.lean,Mathlib/GroupTheory/Commutator/Basic.lean,Mathlib/LinearAlgebra/Basis/Fin.lean,Mathlib/LinearAlgebra/Center.lean,Mathlib/LinearAlgebra/Determinant.lean,Mathlib/LinearAlgebra/Dual/Defs.lean,Mathlib/LinearAlgebra/FiniteDimensional/Basic.lean,Mathlib/LinearAlgebra/FiniteDimensional/Lemmas.lean,Mathlib/LinearAlgebra/LinearIndependent/Lemmas.lean,Mathlib/LinearAlgebra/Projectivization/Action.lean,Mathlib/LinearAlgebra/Projectivization/Basic.lean,Mathlib/LinearAlgebra/SpecialLinearGroup.lean,Mathlib/LinearAlgebra/SpecialLinearGroup/Simple.lean,Mathlib/LinearAlgebra/Transvection.lean,Mathlib/LinearAlgebra/Transvection/Basic.lean,Mathlib/LinearAlgebra/Transvection/Generation.lean,Mathlib/LinearAlgebra/Transvection/SpecialLinearGroup.lean 17 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
0-40999
11 hours ago
unknown
unknown
33693 yoh-tanimoto
author:yoh-tanimoto
feat(Mathlib/Analysis/Normed/Module): add instances of `CompleteSpace` for `Submodules` and `ClosedSubmodule` add an instance of `CompleteSpace` for a `Submodule` of a Banach space `[NormedField 𝕜] [NormedAddCommGroup E] [NormedSpace 𝕜 E] [CompleteSpace E]` which `IsClosed`. ~~In this relation, convert a lemma showing `IsClosed` to an instance for `ClosedSubmodule`.~~ motivation: Together with #28709, this makes it automatic that a `ClosedSubmodule` in a Hilbert space `HasOrthogonalProjection`. discussion: https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/.60CompleteSpace.60.20for.20closed.20subtypes.20in.20a.20.60CompleteSpace.60 19/1 Mathlib/Analysis/InnerProductSpace/Orthogonal.lean,Mathlib/Topology/Algebra/Module/Basic.lean,Mathlib/Topology/Algebra/Module/ClosedSubmodule.lean 3 8 ['github-actions', 'leanprover-radar', 'sgouezel', 'yoh-tanimoto'] jcommelin
assignee:jcommelin
0-38547
10 hours ago
0-45052
12 hours ago
7-17198
7 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` 157/7 Mathlib/Analysis/Convex/Cone/Basic.lean,Mathlib/Analysis/Convex/Cone/Dual.lean,Mathlib/Analysis/InnerProductSpace/Orthogonal.lean,Mathlib/Topology/Algebra/Module/ClosedSubmodule.lean 4 26 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot', 'sgouezel', 'yoh-tanimoto'] sgouezel
assignee:sgouezel
0-35355
9 hours ago
0-33297
9 hours ago
20-60256
20 days
33985 YellPika
author:YellPika
feat(Order/OmegaCompletePartialOrder): `OmegaCompletePartialOrder` instance for `Sum` with basic `ωScottContinuous` lemmas This PR adds an `OmegaCompletePartialOrder` instance for `Sum`, along with `ωScottContinuous` lemmas for basic operations (`inl`, `inr`, `elim`). Appropriate lemmas are marked with `@[fun_prop]` so that the `fun_prop` tactic can automatically deduce `ωScottContinuous` proofs for functions involving `Sum`s (e.g. see the proof of `Sum.ωScottContinuous_map`). - [ ] depends on: #33941 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor large-import blocked-by-other-PR 330/32 Mathlib/Data/Sum/Order.lean,Mathlib/Order/OmegaCompletePartialOrder.lean,Mathlib/Order/ScottContinuity.lean 3 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
0-30812
8 hours ago
0-33532
9 hours ago
0-6
6 seconds

PRs with contradictory labels

There are currently no PRs with contradictory labels. Congratulations!