The mathlib review queue

Welcome to the mathlib review page. Everybody's help with reviewing is appreciated. Reviewing contributions is important, and everybody is welcome to review pull requests! If you're not sure how, the pull request review guide is there to help you.
This page contains tables of

This dashboard was last updated on: August 01, 2025 at 21:39 UTC

Review queue

Number Author Title Description Labels +/- Modified files (first 100) 📝 💬 All users who commented or reviewed Assignee(s) Updated Last status change total time in review
22231 pechersky
author:pechersky
feat(Algebra/Valued): `AdicExpansion` initial defns --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-topology
label:t-algebra$
299/0 Mathlib.lean,Mathlib/Topology/Algebra/Valued/AdicExpansion.lean 2 2 ['Thmoas-Guan', 'github-actions'] nobody
89-65397
2 months ago
158-67039
5 months ago
158-67160
158 days
23758 erdOne
author:erdOne
feat(Topology/Algebra): linearly topologized iff non-archimedian ...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/) large-import t-algebra t-topology
label:t-algebra$
138/3 Mathlib/LinearAlgebra/Span/Basic.lean,Mathlib/Topology/Algebra/LinearTopology.lean 2 21 ['ADedecker', 'AntoineChambert-Loir', 'erdOne', 'github-actions', 'grunweg'] ADedecker and AntoineChambert-Loir
assignee:AntoineChambert-Loir assignee:ADedecker
85-31807
2 months ago
106-4251
3 months ago
116-53065
116 days
23238 YaelDillies
author:YaelDillies
feat: extended floor and ceil My motivation for this is to prove `ENat.toENNReal (⨆ i, f i) = ⨆ i, ENat.toENNReal (f i)` and `ENat.toENNReal (⨅ i, f i) = ⨅ i, ENat.toENNReal (f i)`. Kalle Kytölä independently needs this for his formalisation of statistical physics. From MiscYD --- - [x] depends on: #24781 - [x] depends on: #24782 See #15269 for a past attempt. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
235/0 Mathlib.lean,Mathlib/Algebra/Order/Floor/Extended.lean 2 24 ['YaelDillies', 'b-mehta', 'eric-wieser', 'github-actions', 'kkytola', 'mathlib4-dependent-issues-bot', 'urkud'] nobody
82-6971
2 months ago
82-12922
2 months ago
129-65139
129 days
24184 YaelDillies
author:YaelDillies
feat: `[G : H]` notation for the index of `H : Subgroup G` This is a cute notation which I wrote for FLT. Not sure whether we want it in mathlib nor how to include `relindex` in the picture. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra RFC
label:t-algebra$
5/0 Mathlib/GroupTheory/Index.lean 1 7 ['YaelDillies', 'erdOne', 'github-actions', 'j-loreaux', 'kbuzzard'] nobody
81-63364
2 months ago
81-63364
2 months ago
105-1080
105 days
24829 urkud
author:urkud
fix(Topology/Homotopy): fix name&args order of `comp` `ContinuousMap.Homotopy.hcomp` used name & arguments order that matches Mathlib's category theory conventions, not topology conventions. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology 30/19 Mathlib/Topology/Homotopy/Basic.lean,Mathlib/Topology/Homotopy/Contractible.lean,Mathlib/Topology/Homotopy/Equiv.lean,Mathlib/Topology/Homotopy/Lifting.lean 4 5 ['github-actions', 'grunweg', 'urkud'] nobody
80-53479
2 months ago
80-62119
2 months ago
80-62170
80 days
24533 robertmaxton42
author:robertmaxton42
feat (ULift): conjugation by ULift.up/down, misc cast/heq lemmas * Adds the convenience def `ULift.conj x := `down (f (up x))`, and corresponding basic lemmas * Adds lemmas showing that `ULift.up` and `.down` commute with casts and preserve `HEq`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data 31/0 Mathlib/Data/ULift.lean 1 14 ['eric-wieser', 'github-actions', 'robertmaxton42'] nobody
75-44432
2 months ago
91-44072
2 months ago
91-51983
91 days
22300 chrisflav
author:chrisflav
feat(RingTheory/GoingDown): lift `LTSeries` of primes Inductive version of `Ideal.exists_ideal_lt_liesOver_of_lt`. Co-authored by: Sihan Su Co-authored by: Yi Song --- - [x] depends on: #22299 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
27/0 Mathlib/RingTheory/Ideal/GoingDown.lean 1 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
74-15228
2 months ago
74-15352
2 months ago
74-18813
74 days
24333 xcloudyunx
author:xcloudyunx
feat(Combinatorics/SimpleGraph): cycle graph implementation for generic vertex types The existing `cycleGraph` implementation under Combinatorics/SimpleGraph/Circulant.lean only operates over `Fin n`. This PR implements a cycle graph implementation over any generic vertex type. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-combinatorics 187/0 Mathlib.lean,Mathlib/Combinatorics/SimpleGraph/Cycle.lean 2 29 ['IvanRenison', 'github-actions'] kmill
assignee:kmill
71-73849
2 months ago
99-71406
3 months ago
99-71456
99 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/) t-data 7/4 Mathlib/Data/Finsupp/Pointwise.lean 1 6 ['Paul-Lez', 'eric-wieser', 'github-actions'] nobody
67-16141
2 months ago
109-4439
3 months ago
109-4487
109 days
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/) t-algebraic-geometry 123/0 Mathlib.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Singular/Cusp.lean 2 9 ['Multramate', 'acmepjz', 'erdOne', 'github-actions', 'kckennylau'] nobody
67-6596
2 months ago
72-69397
2 months ago
72-69391
72 days
25153 eric-wieser
author:eric-wieser
feat(Algebra/ModEq): a lemma about `[PMOD (n • p)]` This ultimately didn't end up very useful to me, but I think it's still a nice result. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-number-theory 20/0 Mathlib/Algebra/ModEq.lean 1 3 ['YaelDillies', 'eric-wieser', 'github-actions'] nobody
65-53869
2 months ago
69-19608
2 months ago
69-19588
69 days
24095 lecopivo
author:lecopivo
feat: `fun_prop` for Is(Bounded)LinearMap + notation `fun x ↦L[R] f x` Sets up `fun_prop` for `IsLinearMap` and `IsBoundedLinearMap` also adds notation `fun x ↦ₗ[R] f x` and `fun x ↦L[R] f x` to write bundled versions like lambda function instead of the currently used pointfree notation. large-import t-algebra
label:t-algebra$
352/22 Mathlib.lean,Mathlib/Algebra/Algebra/Bilinear.lean,Mathlib/Algebra/Module/LinearMap/Defs.lean,Mathlib/Algebra/Module/LinearMap/End.lean,Mathlib/Algebra/Module/LinearMap/Pi.lean,Mathlib/Algebra/Module/LinearMap/Prod.lean,Mathlib/Analysis/Normed/Operator/BoundedLinearMaps.lean,scripts/noshake.json 8 22 ['eric-wieser', 'github-actions', 'lecopivo'] nobody
64-12658
2 months ago
64-12658
2 months ago
64-31039
64 days
25337 alreadydone
author:alreadydone
feat(RingTheory): invertible modules and Picard group --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
535/0 Mathlib.lean,Mathlib/RingTheory/Finiteness/Cardinality.lean,Mathlib/RingTheory/PicardGroup.lean,docs/references.bib 4 37 ['alreadydone', 'erdOne', 'github-actions', 'kckennylau'] nobody
60-67721
1 month ago
61-77443
2 months ago
61-77430
61 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 t-topology 509/1 Mathlib.lean,Mathlib/Topology/MetricSpace/BundledFun.lean,Mathlib/Topology/UniformSpace/Ultra/Pseudometrizable.lean 3 8 ['ADedecker', 'fpvandoorn', 'github-actions', 'mathlib4-dependent-issues-bot', 'pechersky'] nobody
52-61573
1 month ago
52-61636
1 month ago
68-7171
68 days
25760 robin-carlier
author:robin-carlier
feat(CategoryTheory/Bicategory): (2,1)-categories and `Pith` This PR introduces a class `IsLocallyGroupoid` on bicategories, asserting that every hom-category has an `IsGroupoid` instance. With this definition, `IsLocallyGroupoid (LocallyDiscrete C)` is correctly inferred. Given a bicategory `B`, we introduce a type alias `Pith B` for `B` (realized as a one-field structure), and we equip it with a `Bicategory` instance where the hom-categories are the cores of the hom-categories of `B`. We show that this bicategory is a (2,1)-category, construct an inclusion pseudo-functor from `Pith B` to `B`, and show that every pseudofunctor from a (2,1)-category to `B` factors through this inclusion. --- We can’t fully state the fact that `(pseudofunctorToPith F).comp (inclusion F)` "is" `F` because #18254 is still not merged. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) --- *This PR continues the work from #25150.* *Original PR: https://github.com/leanprover-community/mathlib4/pull/25150* t-category-theory 191/0 Mathlib.lean,Mathlib/CategoryTheory/Bicategory/LocallyGroupoid.lean 2 1 ['github-actions'] nobody
50-46023
1 month ago
50-46096
1 month ago
50-46078
50 days
25804 erdOne
author:erdOne
feat: `∑ z ∈ L, ‖z - x‖⁻ʳ` converges for lattices `L` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) --- *This PR continues the work from #21673.* *Original PR: https://github.com/leanprover-community/mathlib4/pull/21673* t-analysis 319/0 Mathlib.lean,Mathlib/Algebra/BigOperators/Group/Finset/Disjoint.lean,Mathlib/Algebra/Module/ZLattice/Summable.lean,Mathlib/Order/Disjointed.lean 4 1 ['github-actions'] nobody
50-30057
1 month ago
50-36756
1 month ago
50-36738
50 days
25724 bryangingechen
author:bryangingechen
chore: disable scheduled runs of stale issues workflow There's no point in having this run on schedule while it's still in limbo. --- This also seems to have been [completely broken](https://github.com/leanprover-community/mathlib4/actions/workflows/stale.yml) since #21681, since the search string is too long. Maybe we should just delete this. CI 1/2 .github/workflows/stale.yml 1 1 ['github-actions'] nobody
50-26854
1 month ago
50-63723
1 month ago
50-63704
50 days
25842 mitchell-horner
author:mitchell-horner
feat(Combinatorics/SimpleGraph): define turanDensity Define the Turán density `turanDensity H` of a simple graph `H`: `turanDensity H` is the limit of `extremalNumber n H / n.choose 2` as `n` approaches `∞`. Also prove - the Turán density of a simple graph is well-defined, that is, the limit `extremalNumber n H / n.choose 2` as `n` approaches `∞` exists, - `extremalNumber n H` is asymptotically equivalent to `turanDensity H * n.choose 2` as `n` approaches `∞`. --- - [x] depends on: #19865 - [x] depends on: #20681 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) --- *This PR continues the work from #20171.* *Original PR: https://github.com/leanprover-community/mathlib4/pull/20171* t-combinatorics 210/0 Mathlib.lean,Mathlib/Combinatorics/SimpleGraph/Extremal/Basic.lean,Mathlib/Combinatorics/SimpleGraph/Extremal/TuranDensity.lean,Mathlib/Combinatorics/SimpleGraph/Finite.lean,Mathlib/Data/Sym/Sym2.lean,Mathlib/Order/Monotone/Basic.lean 6 2 ['github-actions', 'mathlib4-dependent-issues-bot'] b-mehta
assignee:b-mehta
49-23821
1 month ago
49-23821
1 month ago
49-28953
49 days
26009 linesthatinterlace
author:linesthatinterlace
feat: Add `Vector`/`List.Vector` equivalence This PR continues the work from #25050. Original PR: https://github.com/leanprover-community/mathlib4/pull/25050 migrated-from-branch 125/17 Mathlib/Data/Vector/Basic.lean,Mathlib/Data/Vector/Defs.lean,Mathlib/Logic/Equiv/Array.lean 3 2 ['github-actions', 'linesthatinterlace'] nobody
45-42381
1 month ago
45-42381
1 month ago
45-44906
45 days
25183 YaelDillies
author:YaelDillies
feat: convolution product on linear maps from a coalgebra to an algebra Construct the ring structure on linear maps `C → A` where `C` is a coalgebra and `A` an algebra, where multiplication is given by `(f * g)(x) = ∑ f x₍₁₎ * g x₍₂₎` in Sweedler notation or ``` | μ | | / \ f * g = f g | | \ / δ | ``` diagrammatically, where `μ` stands for multiplication and `δ` for comultiplication. [Zulip](https://leanprover.zulipchat.com/#narrow/channel/217875-Is-there-code-for-X.3F/topic/.60Mul.60.20instance.20on.20algebra.20homomorphisms.20from.20monoid.20algebra) From Toric Co-authored-by: Michał Mrugała Co-authored-by: Yunzhou Xie --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) toric t-algebra
label:t-algebra$
137/0 Mathlib.lean,Mathlib/RingTheory/Coalgebra/Convolution.lean 2 15 ['YaelDillies', 'erdOne', 'eric-wieser', 'github-actions', 'smorel394'] nobody
44-43509
1 month ago
68-8070
2 months ago
68-11990
68 days
25858 themathqueen
author:themathqueen
feat(RingTheory/Coalgebra/MulOpposite): coalgebra instance for MulOpposite Adding an instance for `Aᵐᵒᵖ` being an `R`-coalgebra when `A` is. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra
label:t-algebra$
112/0 Mathlib.lean,Mathlib/RingTheory/Coalgebra/MulOpposite.lean 2 1 ['github-actions'] nobody
43-85580
1 month ago
48-30979
1 month ago
48-31022
48 days
26154 ADedecker
author:ADedecker
refactor: add refactored APIs for algebraic filter bases This PR continues the work from #18437. Original PR: https://github.com/leanprover-community/mathlib4/pull/18437 t-topology 651/0 Mathlib.lean,Mathlib/Topology/Algebra/FilterBasis.lean,Mathlib/Topology/Algebra/FilterBasisNew.lean,Mathlib/Topology/Algebra/Nonarchimedean/Bases.lean,Mathlib/Topology/Algebra/Nonarchimedean/BasesNew.lean 5 2 ['ADedecker', 'github-actions'] nobody
43-32490
1 month ago
43-32490
1 month ago
43-32548
43 days
26157 erdOne
author:erdOne
chore(RingTheory): Merge `Mathlib/RingTheory/LocalRing/ResidueField/Algebraic.lean` into `Instances.lean` This was added a week ago by myself so I don't think a deprecation is needed --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) file-removed 22/34 Mathlib.lean,Mathlib/NumberTheory/RamificationInertia/Unramified.lean,Mathlib/RingTheory/LocalRing/ResidueField/Algebraic.lean,Mathlib/RingTheory/LocalRing/ResidueField/Instances.lean 4 1 ['github-actions'] nobody
43-28092
1 month ago
43-28253
1 month ago
43-28305
43 days
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/) CI 68/8 .github/build.in.yml,.github/workflows/bors.yml,.github/workflows/build.yml,.github/workflows/build_fork.yml 4 1 ['github-actions'] nobody
42-44054
1 month ago
42-44060
1 month ago
42-44104
42 days
26130 kmill
author:kmill
feat: make `reassoc_of%` be able to defer `Category` instance This PR modifies the elaboration of `reassoc_of%` so that the `Category` instance can be synthesized later, like any other instance metavariable, rather than needing to be synthesized up front, when the category itself might not yet be known. This fixes an issue reported by Robert Maxton [on Zulip](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/reassoc_of.25.20misleading.20error/near/524678383), where in the following `reassoc_of% Sigma.ι_desc` was failing. ```lean import Mathlib.CategoryTheory.Limits.Shapes.Products open CategoryTheory Limits set_option autoImplicit true variable {C : Type u} [Category.{v, u} C] {β : Type w} {f : β → C} [HasCoproduct f] {P : C} (p : (b : β) → f b ⟶ P) (b : β) example {Q : C} (g : P ⟶ Q) : Sigma.ι f b ≫ Sigma.desc p ≫ g = p b ≫ g := by rw [reassoc_of% Sigma.ι_desc] ``` Without this PR, a workaround is writing `reassoc_of% @Sigma.ι_desc`. The PR adds `Lean.Meta.withEnsuringLocalInstance` for temporarily adding a metavariable as a local instance if it can't yet be synthesized. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta 91/20 Mathlib/Lean/Meta/Basic.lean,Mathlib/Tactic/CategoryTheory/IsoReassoc.lean,Mathlib/Tactic/CategoryTheory/Reassoc.lean,MathlibTest/CategoryTheory/Reassoc.lean 4 6 ['github-actions', 'kmill', 'leanprover-bot', 'sgouezel'] nobody
42-2712
1 month ago
43-60003
1 month ago
43-59985
43 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/) t-linter RFC 14/15 Mathlib/Tactic/Linter/CommandStart.lean 1 5 ['github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot'] nobody
41-83268
1 month ago
41-83268
1 month ago
42-1479
42 days
26258 kckennylau
author:kckennylau
feat(Topology): induction for sheafification --- I currently have binary and unary operation, which should be enough for sheaves. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology 62/1 Mathlib/Topology/Sheaves/LocalPredicate.lean 1 1 ['github-actions'] nobody
41-10498
1 month ago
41-10607
1 month ago
41-10668
41 days
26061 kckennylau
author:kckennylau
feat(AlgebraicGeometry): define Projective Space This defines the projective space over a scheme, indexed by an arbitrary type. --- Zulip discussion: [#maths > Projective Space](https://leanprover.zulipchat.com/#narrow/channel/116395-maths/topic/Projective.20Space/with/524057860) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebraic-geometry 63/0 Mathlib.lean,Mathlib/AlgebraicGeometry/ProjectiveSpace.lean 2 14 ['callesonne', 'erdOne', 'github-actions', 'kckennylau'] nobody
41-8373
1 month ago
44-76037
1 month ago
44-76083
44 days
26120 vasnesterov
author:vasnesterov
feat(Data/Seq): `modify` and `set` operations for `Seq` Introduce `modify` and `set` operations for sequences, along with a few lemmas about them. --- - [x] depends on: #20071 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) This PR continues the work from #20160. Original PR: https://github.com/leanprover-community/mathlib4/pull/20160 t-data 69/0 Mathlib/Data/Seq/Seq.lean 1 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'vasnesterov'] nobody
40-25486
1 month ago
44-6822
1 month ago
44-6872
44 days
26284 plp127
author:plp127
feat: faster implementation of `Nat.primeFactorsList` + `@[csimp]` lemma Add a function `Nat.primeFactorsListFast` that `#eval`s faster, and a `@[csimp]` lemma `Nat.primeFactorsList_eq_primeFactorsListFast` that shows `Nat.primeFactorsList = Nat.primeFactorsListFast`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data 95/0 Mathlib/Data/Nat/Factors.lean 1 1 ['github-actions'] nobody
39-61470
1 month ago
39-61493
1 month ago
39-75408
39 days
26301 Ivan-Sergeyev
author:Ivan-Sergeyev
feat(LinearAlgebra/Matrix/Determinant/TotallyUnimodular): Empty matrices are totally unimodular. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra
label:t-algebra$
15/0 Mathlib/LinearAlgebra/Matrix/Determinant/TotallyUnimodular.lean 1 1 ['github-actions'] nobody
39-28860
1 month ago
39-28870
1 month ago
39-28913
39 days
26190 tb65536
author:tb65536
feat(FieldTheory/Galois/IsGaloisGroup): Subgroups of a Galois group are Galois groups This PR gives an instance `IsGaloisGroup H (FixedPoints.intermediateField H : IntermediateField K L) L` from `IsGaloisGroup G K L`, and a numerical corollary. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
11/0 Mathlib/FieldTheory/Galois/IsGaloisGroup.lean 1 1 ['github-actions'] nobody
39-19330
1 month ago
39-19331
1 month ago
42-75331
42 days
26332 Timeroot
author:Timeroot
feat (ModelTheory/Definability): TermDefinable functions This PR continues the work from #23506. Original PR: https://github.com/leanprover-community/mathlib4/pull/23506 large-import 159/0 Mathlib/Data/Rel.lean,Mathlib/ModelTheory/Definability.lean,scripts/noshake.json 3 2 ['Timeroot', 'github-actions'] nobody
38-66915
1 month ago
38-66922
1 month ago
38-66964
38 days
23460 Timeroot
author:Timeroot
feat: Definition of `Clone` Basics about Clones. Part of #20051 --- - [x] depends on: #23459 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
326/0 Mathlib.lean,Mathlib/Algebra/Clone/Basic.lean,Mathlib/Algebra/Clone/Defs.lean,Mathlib/Data/Fin/Basic.lean 4 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
38-66364
1 month ago
38-66366
1 month ago
38-67656
38 days
26462 PSchwahn
author:PSchwahn
feat(LinearAlgebra/Projection): add results about inverse of `Submodule.prodEquivOfIsCompl` Add two theorems `Submodule.prodEquivOfIsCompl_symm_apply` and `Submodule.prodEquivOfIsCompl_symm_add`, which are API for `Submodule.prodEquivOfIsCompl`. We believe these theorems are useful; for example, we have used their statements in a [classification formalization project](https://github.com/LieLean/LowDimSolvClassification). I am not sure whether the `prodEquivOfIsCompl_symm_apply` theorem should be tagged with `@[simp]`; this might lead to confluence issues. Opinions are welcome! Co-authored by: - [Viviana del Barco](https://github.com/vdelbarc) - [Gustavo Infanti](https://github.com/GuQOliveira) - [Exequiel Rivas](https://github.com/erivas) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra
label:t-algebra$
9/0 Mathlib/LinearAlgebra/Projection.lean 1 5 ['PSchwahn', 'github-actions', 'kckennylau'] nobody
33-80619
1 month ago
35-66253
1 month ago
35-66377
35 days
22662 plp127
author:plp127
feat: Localization.Away.lift (computably) This PR adds `Localization.Away.lift'` and `Localization.Away.lift`, computable alternatives to `Localization.awayLift`. --- - [x] depends on: #24791 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
74/0 Mathlib/RingTheory/Localization/Away/Basic.lean 1 12 ['eric-wieser', 'github-actions', 'mathlib4-dependent-issues-bot', 'plp127', 'vihdzp'] nobody
33-56619
1 month ago
81-78702
2 months ago
147-78684
147 days
26510 alreadydone
author:alreadydone
feat(Matroid): exchange lemmas involving closure --- for #24350 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data t-combinatorics 37/0 Mathlib/Data/Matroid/Closure.lean 1 1 ['github-actions'] nobody
33-26285
1 month ago
33-26311
1 month ago
33-26355
33 days
25832 xroblot
author:xroblot
feat(FieldTheory/LinearDisjoint): `trace` (resp. `norm`) and `algebraMap` commutes For `A` and `B` two linearly disjoint `R`-subalgebras in a commutative algebra `S` and `b` a `R`-basis of `B`, we construct a `A`-basis of `S = A ⊔ B` from `b` (and a similar construction using a `R`-basis of `A`). Then, we prove in this situation that `trace` commutes with `algebraMap`, that is: ```lean Algebra.trace A S (algebraMap B S x) = algebraMap R A (Algebra.trace R B x) ``` and a similar result for the norm. We also add a similar basis construction for `A` and `B` two linearly disjoint intermediate fields with the hypothesis that `A.toSubalgebra ⊔ B.toSubalgebra = ⊤`. This hypothesis is equivalent to `A ⊔ B = ⊤` in many cases (for example, one of the two extensions is algebraic over the base field) but not always. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-algebra
label:t-algebra$
161/9 Mathlib/FieldTheory/LinearDisjoint.lean,Mathlib/RingTheory/LinearDisjoint.lean 2 23 ['acmepjz', 'github-actions', 'xroblot'] nobody
32-30613
1 month ago
41-50193
1 month ago
48-81577
48 days
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/) large-import 195/0 Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Monoidal/Basic.lean,Mathlib/CategoryTheory/Enriched/Linear.lean,Mathlib/CategoryTheory/Linear/Basic.lean,Mathlib/CategoryTheory/Monoidal/Linear.lean 5 1 ['github-actions'] nobody
32-26094
1 month ago
38-29478
1 month ago
38-29528
38 days
25947 qawbecrdtey
author:qawbecrdtey
feat(Data/Nat/Factors): added lemmas including `primeFactorsList_length_ne_zero` --- Added lemmas `primeFactorsList_length_ne_zero`, `primeFactorsList_prime_iff`, and `primeFactorsList_length_eq_one`. ```lean theorem primeFactorsList_length_ne_zero (n : ℕ) : n.primeFactorsList.length ≠ 0 ↔ 2 ≤ n theorem primeFactorsList_prime_iff {p : ℕ} : p.primeFactorsList = [p] ↔ p.Prime @[simp] theorem primeFactorsList_length_eq_one (n : ℕ) : n.primeFactorsList.length = 1 ↔ n.Prime ``` [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data 21/3 Mathlib/Data/Nat/Factors.lean 1 5 ['Ruben-VandeVelde', 'github-actions', 'qawbecrdtey'] nobody
31-75294
1 month ago
46-39721
1 month ago
46-48322
46 days
26555 Komyyy
author:Komyyy
feat: lemmas about betweeness on a linear space This PR also adds aliases of the inverse direction of betweeness iff lemmas. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-euclidean-geometry 86/0 Mathlib/Analysis/Convex/Between.lean 1 1 ['github-actions'] nobody
31-69530
1 month ago
32-11125
1 month ago
32-14332
32 days
25843 mitchell-horner
author:mitchell-horner
feat(Combinatorics/SimpleGraph): define `between` subgraphs The simple graph `G.between s t` is the subgraph of `G` containing edges that connect a vertex in the set `s` to a vertex in the set `t`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) --- *This PR continues the work from #24948.* *Original PR: https://github.com/leanprover-community/mathlib4/pull/24948* t-combinatorics 95/0 Mathlib/Combinatorics/SimpleGraph/Bipartite.lean 1 1 ['github-actions'] nobody
31-6499
1 month ago
49-28673
1 month ago
49-28656
49 days
25758 YaelDillies
author:YaelDillies
chore: shortcut instance `CompleteLattice α → PartialOrder α` This avoids using the path `CompleteLattice α → CompletePartialOrder α → PartialOrder α` that goes through `Order.CompletePartialOrder` and makes it appear used to our automation, such as `shake` or `#min_imports`. This is a followup to #25358. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order 7/0 Mathlib/Order/CompleteLattice/Defs.lean 1 6 ['Ruben-VandeVelde', 'eric-wieser', 'github-actions', 'leanprover-bot'] nobody
30-80037
30 days ago
30-82062
30 days ago
50-46246
50 days
26563 winstonyin
author:winstonyin
chore: rename `IsIntegralCurve` to `IsMIntegralCurve` I rename all the existing `IsIntegralCurve` series of definitions and lemmas for manifolds to `IsMIntegralCurve` in preparation for reusing `IsIntegralCurve` for the vector space version. - [ ] depends on: #26533 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-differential-geometry 320/165 Mathlib/Geometry/Manifold/IntegralCurve/Basic.lean,Mathlib/Geometry/Manifold/IntegralCurve/ExistUnique.lean,Mathlib/Geometry/Manifold/IntegralCurve/Transform.lean,Mathlib/Geometry/Manifold/IntegralCurve/UniformTime.lean,docs/overview.yaml 5 8 ['github-actions', 'grunweg', 'mathlib4-dependent-issues-bot', 'winstonyin'] grunweg
assignee:grunweg
29-81935
29 days ago
29-82114
29 days ago
30-35135
30 days
23986 ShouxinZhang
author:ShouxinZhang
feat(FieldTheory/RatFunc): add RatFunc.toFractionRingAlgEquiv --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra
label:t-algebra$
13/0 Mathlib/FieldTheory/RatFunc/Basic.lean 1 32 ['ShouxinZhang', 'eric-wieser', 'github-actions', 'joneugster', 'kckennylau', 'plp127'] nobody
29-75617
29 days ago
32-2073
1 month ago
110-65010
110 days
26148 Hagb
author:Hagb
feat(RingTheory/Ideal/Span): some lemmas about zero and span `simp` would be able to solve them. Notice that `span_singleton_zero : span {(0 : R)} = ⊥` itself can be solved by `simp` without this commit, which uses `span_singleton_eq_bot : span ({x} : Set α) = ⊥ ↔ x = 0`, while `simp` cannot solve goals like `f (Ideal.span {(0 : R)}) = f ⊥`, which would be solvable by `simp` with `span_singleton_zero` marked with `@[simp]`. Without adding also `Ideal.dvd_bot`, these lemmas on `Span.lean` would make the following failed, since `simp` would rewrite `{0}` with `⊥` and result in a goal `v.asIdeal ∣ ⊥` that it can't solve. https://github.com/leanprover-community/mathlib4/blob/3f2556372f27171259a381d4d57db71440700cd8/Mathlib/RingTheory/DedekindDomain/AdicValuation.lean#L123 --- This PR continues the work from #24448. Original PR: #24448. CC: @tb65536 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) migrated-from-branch t-algebra
label:t-algebra$
11/0 Mathlib/RingTheory/Ideal/Operations.lean,Mathlib/RingTheory/Ideal/Span.lean 2 1 ['github-actions'] nobody
29-52751
29 days ago
29-52751
29 days ago
43-38269
43 days
22039 YaelDillies
author:YaelDillies
feat: simproc for computing `Finset.Ixx` of natural numbers --- - [x] depends on: #22290 - [x] depends on: #22559 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-meta 315/0 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Simproc/FinsetInterval.lean,Mathlib/Util/Qq.lean 4 59 ['FLDutchmann', 'Paul-Lez', 'YaelDillies', 'eric-wieser', 'github-actions', 'grunweg', 'kim-em', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'urkud'] eric-wieser
assignee:eric-wieser
29-27643
29 days ago
107-41026
3 months ago
163-1744
163 days
26313 kckennylau
author:kckennylau
feat: 4 lemmas about Finsupp.mapDomain.linearEquiv --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
9/0 Mathlib/LinearAlgebra/Finsupp/Defs.lean 1 5 ['eric-wieser', 'github-actions', 'kckennylau'] nobody
29-17847
29 days ago
39-19368
1 month ago
39-19418
39 days
25692 Whysoserioushah
author:Whysoserioushah
feat(RingTheory/MatrixAlgebra): add a more general version of `matrixEquivTensor` This adds `tensorMatrixLinearEquiv : A ⊗[R] Matrix n n B ≃ₐ[S] Matrix n n (A ⊗[R] B)` which is a more general version of `matrixEquivTensor : Matrix n n A ≃ₐ[R] (A ⊗[R] Matrix n n R)`. The latter is then implemented as a trivial consequence of the former. Many internal implementation details are deleted without deprecation, although strictly these were not `private. Co-authored-by: @erdOne Co-authored-by: Eric Wieser --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
122/100 Mathlib/Data/Matrix/Basis.lean,Mathlib/RingTheory/MatrixAlgebra.lean 2 13 ['Whysoserioushah', 'eric-wieser', 'github-actions'] nobody
29-2480
29 days ago
34-73368
1 month ago
51-42770
51 days
26670 yu-yama
author:yu-yama
feat(GroupExtension/Abelian): define `conjClassesEquivH1` This PR continues the work from #21837. Original PR: https://github.com/leanprover-community/mathlib4/pull/21837 t-algebra
label:t-algebra$
162/5 Mathlib.lean,Mathlib/GroupTheory/GroupExtension/Abelian.lean,Mathlib/GroupTheory/GroupExtension/Basic.lean,Mathlib/GroupTheory/GroupExtension/Defs.lean,docs/references.bib 5 2 ['erdOne', 'github-actions', 'yu-yama'] nobody
28-80141
28 days ago
29-22246
29 days ago
29-22297
29 days
26710 metakunt
author:metakunt
feat (Data/Nat/Digits/Lemmas): Add digits_getD Adds digits_getD, an explicit computation of the i-th digits of n in base b representation. t-data new-contributor 64/0 Mathlib/Data/Nat/Digits/Lemmas.lean 1 1 ['github-actions'] nobody
28-77564
28 days ago
28-77695
28 days ago
28-77746
28 days
25812 vlad902
author:vlad902
feat(data): List.Chain' helper lemmas Add two helpers lemmas to go from a List.Chain' hypothesis to a concrete predicate about two consecutive elements, one in the positive and one in the negative. t-data 29/0 Mathlib/Data/List/Chain.lean 1 4 ['BoltonBailey', 'github-actions', 'vlad902'] nobody
28-58432
28 days ago
29-46726
29 days ago
42-49313
42 days
26267 vasnesterov
author:vasnesterov
feat(Analysis/Calculus): Taylor series converges to function on whole ball * Prove `FormalMultilinearSeries.AnalyticOnNhd`: the sum of series is analytic on its ball of convergence. * Prove `AnalyticOn.hasFPowerSeriesOnBall`: a variant of `AnalyticAt.hasFPowerSeriesAt` which gives convergence to the function on the ball of convergence. --- - [x] depends on: #23745 - [x] depends on: #23747 - [x] depends on: #23748 - [x] depends on: #26247 This PR continues the work from #23749. Original PR: https://github.com/leanprover-community/mathlib4/pull/23749 large-import t-analysis 47/0 Mathlib/Analysis/Analytic/ChangeOrigin.lean,Mathlib/Analysis/Calculus/IteratedDeriv/Lemmas.lean 2 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'vasnesterov'] nobody
28-56977
28 days ago
28-66473
28 days ago
28-72786
28 days
26766 MichaelStollBayreuth
author:MichaelStollBayreuth
feat(Topology/MetricSpace/Bounded): add some results We add two pairs of results: ```lean lemma isBounded_of_abs_le (C : α) : Bornology.IsBounded {x : α | |x| ≤ C} := ... lemma isBounded_of_abs_lt (C : α) : Bornology.IsBounded {x : α | |x| < C} := ... ``` (under suitable assumptions on `α`) and a version of the *Extreme Value Theorem* that I found convenient: ```lean theorem exists_forall_le_of_isBounded {f : β → α} (hf : Continuous f) (x₀ : β) (h : Bornology.IsBounded {x : β | f x ≤ f x₀}) : ∃ x, ∀ y, f x ≤ f y := ... theorem exists_forall_ge_of_isBounded {f : β → α} (hf : Continuous f) (x₀ : β) (h : Bornology.IsBounded {x : β | f x₀ ≤ f x}) : ∃ x, ∀ y, f y ≤ f x := ... ``` (under suitable assumptions on `α` and `β`). For an application, see [GelfandMazur.lean](https://github.com/MichaelStollBayreuth/Heights/blob/master/Heights/GelfandMazur.lean) in [Heights](https://github.com/MichaelStollBayreuth/Heights/tree/master). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology 56/0 Mathlib/Topology/MetricSpace/Bounded.lean 1 1 ['github-actions'] nobody
28-7971
28 days ago
28-7971
28 days ago
28-7953
28 days
19872 YaelDillies
author:YaelDillies
chore(GroupTheory/Index): rename `relindex` to `relIndex` --- - [x] depends on: #24044 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) FLT t-algebra
label:t-algebra$
257/194 Mathlib/FieldTheory/Relrank.lean,Mathlib/GroupTheory/Commensurable.lean,Mathlib/GroupTheory/CosetCover.lean,Mathlib/GroupTheory/GroupAction/Blocks.lean,Mathlib/GroupTheory/Index.lean,Mathlib/GroupTheory/IndexNormal.lean,Mathlib/GroupTheory/PGroup.lean,Mathlib/GroupTheory/Schreier.lean,Mathlib/GroupTheory/SchurZassenhaus.lean,Mathlib/GroupTheory/Sylow.lean,Mathlib/GroupTheory/Transfer.lean,Mathlib/LinearAlgebra/FreeModule/Finite/CardQuotient.lean,Mathlib/NumberTheory/ModularForms/CongruenceSubgroups.lean,Mathlib/NumberTheory/NumberField/Discriminant/Different.lean,Mathlib/NumberTheory/NumberField/Units/Regulator.lean,Mathlib/RingTheory/Ideal/Quotient/Index.lean 16 24 ['Ruben-VandeVelde', 'TwoFX', 'YaelDillies', 'alreadydone', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'loefflerd', 'madvorak', 'mathlib4-dependent-issues-bot', 'tb65536'] nobody
27-53213
27 days ago
27-55795
27 days ago
182-6724
182 days
25732 robin-carlier
author:robin-carlier
feat(CategoryTheory/Monoidal/Limits): miscellany about preservation of (co)limits by tensor products Register some instances regarding preservations of (co)limits for the tensor product of a monoidal category. More precisely, we register the fact that if the category is braided and `tensorLeft c` preserves colimits (this can be inferred e.g via `MonoidalClosed C`), then so does `tensorRight c` for every `c`. We also rephrase preservation of (co)limits for `curriedTensor C` in terms of preservations of (co)limits for `tensorRight c`. The PR introduces also introduces a directory `CategoryTheory.Monoidal.Limits` and moves the existing file `CategoryTheory.Monoidal.Limits.lean` to `CategoryTheory.Monoidal.Limits.Basic`. --- The instances registered here are tailored so that for a braided monoidal closed category, `PreservesColimit₂` instances from #24685 can be inferred with the results of #24686 for the external product of diagrams defined in #24703 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) --- *This PR continues the work from #24711.* *Original PR: https://github.com/leanprover-community/mathlib4/pull/24711* file-removed t-category-theory 72/2 Mathlib.lean,Mathlib/CategoryTheory/Monoidal/Internal/Limits.lean,Mathlib/CategoryTheory/Monoidal/Limits/Basic.lean,Mathlib/CategoryTheory/Monoidal/Limits/Preserves.lean 4 2 ['github-actions', 'leanprover-community-bot-assistant'] nobody
27-53041
27 days ago
27-53059
27 days ago
50-42243
50 days
22655 YaelDillies
author:YaelDillies
refactor: make use of `FunLike` for `Submonoid.LocalizationMap` From Toric --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) toric t-algebra
label:t-algebra$
161/146 Mathlib/GroupTheory/MonoidLocalization/Away.lean,Mathlib/GroupTheory/MonoidLocalization/Basic.lean,Mathlib/GroupTheory/MonoidLocalization/DivPairs.lean,Mathlib/GroupTheory/MonoidLocalization/MonoidWithZero.lean,Mathlib/RingTheory/Localization/Defs.lean,Mathlib/RingTheory/Valuation/ExtendToLocalization.lean 6 4 ['github-actions', 'leanprover-community-bot-assistant'] ericrbg
assignee:ericrbg
27-52576
27 days ago
27-52598
27 days ago
144-43216
144 days
26110 YaelDillies
author:YaelDillies
feat: sharp monoids Define sharp monoids, which are the monoids whose only unit is `1`. This concept is useful in log geometry and in particular shows up in the theory of affine monoids. This concept already existed in the guise of `Subsingleton Mˣ`, but giving it a name makes it easier to refer to and uncovers some missing instances. From Toric --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) toric t-algebra
label:t-algebra$
51/30 Mathlib/Algebra/BigOperators/Associated.lean,Mathlib/Algebra/BigOperators/Group/Finset/Basic.lean,Mathlib/Algebra/GCDMonoid/Basic.lean,Mathlib/Algebra/Group/Irreducible/Defs.lean,Mathlib/Algebra/Group/Pi/Units.lean,Mathlib/Algebra/Group/Prod.lean,Mathlib/Algebra/Group/Submonoid/Units.lean,Mathlib/Algebra/Group/Units/Basic.lean,Mathlib/Algebra/Group/Units/Defs.lean,Mathlib/Algebra/GroupWithZero/Associated.lean,Mathlib/Algebra/GroupWithZero/Divisibility.lean,Mathlib/Data/List/Prime.lean,Mathlib/Data/ZMod/Basic.lean,Mathlib/NumberTheory/DirichletCharacter/Basic.lean,Mathlib/RingTheory/ChainOfDivisors.lean,Mathlib/RingTheory/IntegralDomain.lean,Mathlib/RingTheory/UniqueFactorizationDomain/NormalizedFactors.lean,Mathlib/RingTheory/Valuation/Integers.lean 18 2 ['b-mehta', 'github-actions', 'leanprover-community-bot-assistant'] nobody
27-52011
27 days ago
27-57291
27 days ago
44-16941
44 days
26021 vasnesterov
author:vasnesterov
feat(Data/Real): representation of reals from `[0, 1]` in positional system * Introduce `ofDigits {b : ℕ} (digits : ℕ → Fin b) : ℝ`, representing a real number of the form `0.d₀d₁d₂...` (where `dᵢ = digits i`) as an infinite sum. * Prove that this sum converges to a number in the interval `[0, 1]`. * Prove `ofDigits_close_of_common_prefix`: if the first `n` digits of two numbers are equal, then their difference is bounded by `b⁻ⁿ`. * Introduce `Real.digits`, which converts a real number into its sequence of digits. * Prove that `ofDigits (toDigits x b) = x`. [Zulip thread](https://leanprover.zulipchat.com/#narrow/stream/217875-Is-there-code-for-X.3F/topic/Base.20n.20expansion.20of.20real.20numbers.3F/near/502937293) --- - [x] depends on: #26004 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data 238/0 Mathlib.lean,Mathlib/Data/Real/OfDigits.lean,scripts/noshake.json 3 11 ['alreadydone', 'eric-wieser', 'github-actions', 'mathlib4-dependent-issues-bot', 'vasnesterov', 'wwylele'] nobody
27-50081
27 days ago
30-64849
30 days ago
30-65407
30 days
26057 YaelDillies
author:YaelDillies
feat: `mon_tauto`, a simp set to prove tautologies about a monoid object This simp set proves all tautologies involving (commutative) monoid objects in a (braided) monoidal category. The general algorithm it follows is to push the associators `α_` and commutators `β_` inwards until they cancel against the right sequence of multiplications. This approach is justified by the fact that a tautology in the language of (commutative) monoid objects "remembers" how it was proved: Every use of a (commutative) monoid object axiom inserts a unitor, associator or commutator, and proving a tautology simply amounts to undoing those moves as prescribed by the presence of unitors, associators and commutators in its expression. This simp set is opiniated about its normal form and therefore cannot be used concurrently to some of the simp lemmas in the standard simp set. As an example, we prove `tensorμ M M M M ≫ (μ ⊗ₘ μ) ≫ μ = (μ ⊗ₘ μ) ≫ μ`, the categorical equivalent of `mul_mul_mul_comm`. From Toric Co-authored-by: Andrew Yang --- - [x] depends on: #26102 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) toric t-category-theory 151/1 Mathlib/CategoryTheory/Monoidal/Mon_.lean,Mathlib/Tactic/Attr/Register.lean,MathlibTest/CategoryTheory/Monoidal/MonTauto.lean,scripts/noshake.json 4 11 ['YaelDillies', 'erdOne', 'github-actions', 'mathlib4-dependent-issues-bot', 'robin-carlier'] nobody
27-49800
27 days ago
44-6775
1 month ago
44-69630
44 days
25779 robin-carlier
author:robin-carlier
feat(CategoryTheory/Bicategory/NaturalTransformations): strong and lax natural transformations of lax functors Given two lax functors `F G` between bicategories, we define lax natural transformations as families of 1-morphisms `∀ a : B, F.obj a ⟶ G.obj a` equipped with a naturality 2-cell `∀ {a b : B} (f : a ⟶ b), app a ≫ G.map f ⟶ F.map f ≫ app b` that are required to satisfy conditions such as naturality, and compatibility with the `mapId` and `mapComp` fields of the source and target functors. This notion dualizes the existing notion of oplax natural transformations between, and tries to narrow the current gap between lax and oplax functors in the library, where the latter has much more formalized API. For maintainability, The code tries to stay as aligned as possible with the code in `CategoryTheory.Bicategory.Naturaltransformations.Oplax`. --- I followed the book by Johnson and Yau for the definition. I made @yuma-mizuno and @callesonne authors of the files, as they are the authors of the original code for Oplax functors, which I basically copy-pasted and modified to make it work with lax functors. They should feel free to modify this if they want. Next thing on the list is to tackle modifications between lax/strong natural transforms of lax transforms, as well as the category instance on lax functors. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) --- *This PR continues the work from #25565.* *Original PR: https://github.com/leanprover-community/mathlib4/pull/25565* t-category-theory 286/0 Mathlib.lean,Mathlib/CategoryTheory/Bicategory/NaturalTransformation/Lax.lean,scripts/noshake.json 3 3 ['github-actions', 'yuma-mizuno'] nobody
27-49500
27 days ago
27-49545
27 days ago
49-7912
49 days
22151 alreadydone
author:alreadydone
feat(RingTheory): a semiprimary ring is Noetherian/Artinian iff its Jacobson radical is fg A key fact used is `Module.FG.smul`: if `I` is a two-sided ideal of `R` that is f.g. as a left ideal and `N` is a f.g. `R`-module, then `I • M` is also a f.g. `R`-module. Many lemmas about coprimality of ideals are also generalized to the noncommutative, two-sided setting. --- - [x] depends on: #21904 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
217/157 Mathlib/Algebra/Algebra/Operations.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Affine/Point.lean,Mathlib/NumberTheory/RamificationInertia/Basic.lean,Mathlib/RingTheory/Extension/Basic.lean,Mathlib/RingTheory/Finiteness/Basic.lean,Mathlib/RingTheory/Finiteness/Ideal.lean,Mathlib/RingTheory/HopkinsLevitzki.lean,Mathlib/RingTheory/Ideal/Maps.lean,Mathlib/RingTheory/Ideal/Operations.lean 9 8 ['alreadydone', 'github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
27-3862
27 days ago
27-7044
27 days ago
149-43846
149 days
26547 robin-carlier
author:robin-carlier
feat(CategoryTheory/Limits/Shapes/Pullback/Categorical/CatCospanTransform): more lemmas about isomorphisms of `CatCospanTransform` We construct ways to extract left, right or base components of ismorphisms of `CatCospanTransform`, as well as various `IsIso` instances, and lemmas allowing to compute the left, right or base component of the inverse of a `CatCospanTransformMorphism` that has an `IsIso` instance. --- - [x] depends on: #26412 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory 70/0 Mathlib/CategoryTheory/Limits/Shapes/Pullback/Categorical/CatCospanTransform.lean 1 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
26-50690
26 days ago
27-43859
27 days ago
27-46905
27 days
24719 madvorak
author:madvorak
feat(LinearAlgebra/Matrix/NonsingularInverse): inverting `Matrix` inverts its `LinearEquiv` --- Discussion: https://leanprover.zulipchat.com/#narrow/channel/144837-PR-reviews/topic/.2324719.20cannot.20find.20home/with/517142655 t-algebra
label:t-algebra$
10/0 Mathlib/LinearAlgebra/Matrix/NonsingularInverse.lean 1 15 ['eric-wieser', 'github-actions', 'madvorak'] nobody
26-45385
26 days ago
82-30574
2 months ago
83-66800
83 days
26746 alreadydone
author:alreadydone
feat(RingTheory): integral extensions of comm. rings are local homs migrated from #23684 --- The import increase only affects one file so I hope it's okay. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import 59/66 Mathlib/Algebra/Field/Equiv.lean,Mathlib/Algebra/Group/Invertible/Basic.lean,Mathlib/Algebra/GroupWithZero/Units/Basic.lean,Mathlib/AlgebraicGeometry/Morphisms/Proper.lean,Mathlib/FieldTheory/LinearDisjoint.lean,Mathlib/LinearAlgebra/Dimension/Localization.lean,Mathlib/NumberTheory/RamificationInertia/Unramified.lean,Mathlib/RingTheory/Artinian/Ring.lean,Mathlib/RingTheory/Ideal/Int.lean,Mathlib/RingTheory/IntegralClosure/Algebra/Defs.lean,Mathlib/RingTheory/IntegralClosure/IsIntegralClosure/Basic.lean,Mathlib/RingTheory/LinearDisjoint.lean,Mathlib/RingTheory/Localization/FractionRing.lean,Mathlib/RingTheory/Localization/Integral.lean,Mathlib/RingTheory/SimpleRing/Field.lean 15 7 ['alreadydone', 'github-actions', 'leanprover-bot', 'mariainesdff'] mariainesdff
assignee:mariainesdff
26-42852
26 days ago
26-42852
26 days ago
28-26415
28 days
26607 vihdzp
author:vihdzp
feat(SetTheory/Cardinal/Aleph): characterization of initial successor ordinals --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-set-theory 5/0 Mathlib/SetTheory/Cardinal/Aleph.lean 1 5 ['github-actions', 'kckennylau', 'vihdzp'] nobody
26-25843
26 days ago
30-70399
30 days ago
30-70443
30 days
26770 Jun2M
author:Jun2M
feat(Combinatorics/Graph) : subgraph relations and operations on `Graph` This PR creates a new file `Combinatorics/Graph/Subgraph.lean`. In it, the PR introduces a partial order on graphs by subgraph relation, defines relations `IsInducedSubgraph`, `IsSpanningSubgraph` and `IsClosedSubgraph`. Further, it introduce operations `EdgeRestrict`, `EdgeDelete`, `induce` and `VertexDelete`. Co-authored-by: Peter Nelson --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics 703/0 Mathlib.lean,Mathlib/Combinatorics/Graph/Subgraph.lean 2 1 ['github-actions'] nobody
26-10574
26 days ago
27-85788
27 days ago
27-85831
27 days
26829 pechersky
author:pechersky
feat(RingTheory/Valuation): Valuation.leAddSubgroup and ideal/submodule versions of ltAddSubgroup Extracted from #25450 without changing how Valued works --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) @faenuccio hopefully this bypasses any wait on #14752 because I am not changing Valued files. t-algebra
label:t-algebra$
177/0 Mathlib/RingTheory/Valuation/Basic.lean,Mathlib/RingTheory/Valuation/Integers.lean 2 1 ['github-actions'] nobody
25-83083
25 days ago
26-2201
26 days ago
26-2255
26 days
26822 jsm28
author:jsm28
feat(LinearAlgebra/AffineSpace): affine combinations and spans of images Add two lemmas about affine combinations and the spans of points in a subset of an indexed family. ```lean /-- A point in the `affineSpan` of a subset of an indexed family is an `affineCombination` with sum of weights 1, using only points in the given subset. -/ lemma eq_affineCombination_of_mem_affineSpan_image {p₁ : P} {p : ι → P} {s : Set ι} (h : p₁ ∈ affineSpan k (p '' s)) : ∃ (fs : Finset ι) (w : ι → k), ↑fs ⊆ s ∧ ∑ i ∈ fs, w i = 1 ∧ p₁ = fs.affineCombination k p w := by ``` ```lean /-- If an affine combination of affinely independent points lies in the affine span of a subset of those points, all weights outside that subset are zero. -/ lemma AffineIndependent.eq_zero_of_affineCombination_mem_affineSpan {p : ι → P} (ha : AffineIndependent k p) {fs : Finset ι} {w : ι → k} (hw : ∑ i ∈ fs, w i = 1) {s : Set ι} (hm : fs.affineCombination k p w ∈ affineSpan k (p '' s)) {i : ι} (hifs : i ∈ fs) (his : i ∉ s) : w i = 0 := by ``` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
27/0 Mathlib/LinearAlgebra/AffineSpace/Combination.lean,Mathlib/LinearAlgebra/AffineSpace/Independent.lean 2 1 ['github-actions'] nobody
25-76761
25 days ago
26-14001
26 days ago
26-13983
26 days
25776 Parcly-Taxel
author:Parcly-Taxel
chore: deprime `induction` in `Analysis` I think this is very marginally dependent on #25770. tech debt t-analysis 256/208 Mathlib/Analysis/Analytic/Composition.lean,Mathlib/Analysis/Analytic/Constructions.lean,Mathlib/Analysis/Analytic/Inverse.lean,Mathlib/Analysis/BoxIntegral/Basic.lean,Mathlib/Analysis/BoxIntegral/Box/SubboxInduction.lean,Mathlib/Analysis/BoxIntegral/Partition/Additive.lean,Mathlib/Analysis/BoxIntegral/Partition/Split.lean,Mathlib/Analysis/CStarAlgebra/Basic.lean,Mathlib/Analysis/CStarAlgebra/Multiplier.lean,Mathlib/Analysis/Calculus/ContDiff/Basic.lean,Mathlib/Analysis/Calculus/ContDiff/Bounds.lean,Mathlib/Analysis/Calculus/ContDiff/FTaylorSeries.lean,Mathlib/Analysis/Calculus/ContDiff/Operations.lean,Mathlib/Analysis/Calculus/Deriv/ZPow.lean,Mathlib/Analysis/Calculus/InverseFunctionTheorem/ApproximatesLinearOn.lean,Mathlib/Analysis/Calculus/IteratedDeriv/Lemmas.lean,Mathlib/Analysis/Calculus/SmoothSeries.lean,Mathlib/Analysis/Convex/Combination.lean,Mathlib/Analysis/Convex/Radon.lean,Mathlib/Analysis/InnerProductSpace/Projection.lean,Mathlib/Analysis/Normed/Algebra/Exponential.lean,Mathlib/Analysis/NormedSpace/Multilinear/Basic.lean,Mathlib/Analysis/Seminorm.lean,Mathlib/Analysis/SpecialFunctions/Complex/Arg.lean,Mathlib/Analysis/SpecialFunctions/Complex/Circle.lean,Mathlib/Analysis/SpecialFunctions/Gamma/Basic.lean,Mathlib/Analysis/SpecialFunctions/Gamma/Beta.lean,Mathlib/Analysis/SpecialFunctions/Gamma/BohrMollerup.lean,Mathlib/Analysis/SpecialFunctions/Gamma/Deriv.lean,Mathlib/Analysis/SpecialFunctions/Integrals/Basic.lean,Mathlib/Analysis/SpecialFunctions/Log/Basic.lean,Mathlib/Analysis/SpecialFunctions/Pow/Deriv.lean,Mathlib/Analysis/SpecialFunctions/Pow/NNReal.lean,Mathlib/Analysis/SpecialFunctions/Pow/Real.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/EulerSineProd.lean 35 3 ['Parcly-Taxel', 'github-actions', 'leanprover-community-bot-assistant', 'madvorak'] nobody
25-39140
25 days ago
25-73112
25 days ago
48-53287
48 days
25830 ScottCarnahan
author:ScottCarnahan
refactor (RingTheory/HahnSeries/HEval): remove positive order condition from definition This PR removes the positive order condition for substitution (or Hahn evaluation) of a Hahn series into a power series. When the order is not positive, the function substitutes zero. We also add short lemmas for substitution into `PowerSeries.X` and `PowerSeries.C`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) --- *This PR continues the work from #24498.* *Original PR: https://github.com/leanprover-community/mathlib4/pull/24498* t-algebra
label:t-algebra$
34/15 Mathlib/RingTheory/HahnSeries/HEval.lean 1 2 ['github-actions', 'leanprover-community-bot-assistant'] nobody
23-45431
23 days ago
25-12017
25 days ago
47-15685
47 days
26814 KiringYJ
author:KiringYJ
feat(MeasureTheory): expose `m.SigmaAlgebra` and `IsSigmaAlgebra` (New PR opened because I mis-clicked “Merge” on the previous branch and had to revert it.) This PR introduces a lightweight API for treating the σ‑algebra of a `MeasurableSpace` as a plain `Set (Set α)`, plus a semantic predicate `IsSigmaAlgebra` and small bridges between bundled and un‑bundled views. #### Motivation The immediate goal is to prepare for a formalization of the **monotone class theorem**. With `m.SigmaAlgebra` and the `IsSigmaAlgebra` predicate, one can state the theorem as a clean equality of families of sets, e.g. ```lean SigmaAlgebra.generateFrom G = MonotoneClass.generateFrom G ``` rather than the more cumbersome phrasing "`s` is measurable ↔ `s` belongs to the smallest monotone class containing `G`". The helpers in this PR make those equalities ergonomic and reusable. #### What’s new - **`m.SigmaAlgebra`** – the collection of all `m`‑measurable sets, exposed as a value of type `Set (Set α)`. Lets you write `s ∈ m.SigmaAlgebra` instead of `MeasurableSet[m] s`. - **`IsSigmaAlgebra F`** – predicate saying that a family of sets `A` is already a σ‑algebra, defined by `(generateFrom F).SigmaAlgebra = F`. - **`generateFrom_sigmaAlgebra_eq`** – idempotence lemma `generateFrom m.SigmaAlgebra = m` (`@[simp]`). - Boolean‑algebra instance on `m.SigmaAlgebra` (alias of the existing subtype instance). - Helper lemmas: - `Subtype.mem_sigma` – bundled measurable set ∈ `m.SigmaAlgebra`. - `Set.toMeasurableSubtype` – wrap a membership proof into the subtype. #### House‑keeping - Removed two obsolete `noncomputable` keywords from `Mathlib/MeasureTheory/MeasurablyGenerated.lean`; the affected instances are now computable. #### Notes - **No breaking changes**: the new definitions are additive; existing code continues to compile unchanged. - **No dependencies on other PRs**: this patch is self‑contained. new-contributor t-measure-probability 86/3 Mathlib.lean,Mathlib/MeasureTheory/MeasurableSpace/MeasurablyGenerated.lean,Mathlib/MeasureTheory/MeasurableSpace/SigmaAlgebra.lean 3 1 ['github-actions'] nobody
22-56765
22 days ago
26-45734
26 days ago
26-45778
26 days
26881 emo916math
author:emo916math
feat(Analysis/Calculus/Deriv/Star) A formula for `deriv (conj ∘ f ∘ conj)` Added a lemma that `deriv (conj ∘ f ∘ conj) = conj ∘ deriv f ∘ conj`, proved by cases on whether the derivative mathematically exists or not. This PR replaces [#26805](https://github.com/leanprover-community/mathlib4/pull/26805); see discussion there. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-analysis 50/2 Mathlib/Analysis/Calculus/Deriv/Star.lean 1 7 ['emo916math', 'github-actions', 'kckennylau'] nobody
22-8646
22 days ago
25-5684
25 days ago
25-5728
25 days
26022 AntoineChambert-Loir
author:AntoineChambert-Loir
feat(RingTheory/MvPolynomial/Groebner): add docstring and a particular case * add a new division theorem when one divides by a single polynomial * add docstrings to the three division theorems This PR continues the work from #24819. Original PR: https://github.com/leanprover-community/mathlib4/pull/24819 t-algebra
label:t-algebra$
27/3 Mathlib/RingTheory/MvPolynomial/Groebner.lean 1 2 ['AntoineChambert-Loir', 'github-actions'] nobody
21-81414
21 days ago
45-35081
1 month ago
45-35130
45 days
26988 YaelDillies
author:YaelDillies
feat(Rel): more API Some of this API already exists in `Topology.UniformSpace.Defs` but not spelled with `Rel`, some of it was written for #24173. --- `Topology.UniformSpace.Defs` will be refactored to use these new lemmas in #23181. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data 169/7 Mathlib/Combinatorics/SimpleGraph/Basic.lean,Mathlib/Data/Rel.lean 2 1 ['github-actions'] nobody
21-36255
21 days ago
21-40080
21 days ago
21-40131
21 days
27000 gasparattila
author:gasparattila
feat(Analysis/Normed/Group/Quotient): isometric versions of isomorphisms This PR adds an isometric version of the third isomorphism theorem for groups and modules. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import new-contributor t-analysis 49/2 Mathlib/Analysis/Normed/Group/Quotient.lean 1 1 ['github-actions'] nobody
21-27046
21 days ago
21-27048
21 days ago
21-27100
21 days
27019 Komyyy
author:Komyyy
feat: T1 Alexandrov-discrete topology is discrete --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology 24/0 Mathlib.lean,Mathlib/Topology/Separation/AlexandrovDiscrete.lean 2 1 ['github-actions'] nobody
20-59102
20 days ago
20-59404
20 days ago
20-59388
20 days
26838 vlad902
author:vlad902
feat: add lemmas about `List.scanr` This PR continues the work from #25188. Original PR: https://github.com/leanprover-community/mathlib4/pull/25188 t-data 84/19 Mathlib/Data/List/Scan.lean 1 12 ['github-actions', 'vihdzp', 'vlad902'] nobody
20-48946
20 days ago
25-51455
25 days ago
25-51508
25 days
27030 YaelDillies
author:YaelDillies
refactor: use `Algebra.FiniteType` as a class Assumptions are currently being passed explicitly, which is quite odd. Also generalise the ~lemmas~ instances about `Polynomial`, `MvPolynomial`, etc... to be about two rings instead of one. From Toric --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) toric t-algebra
label:t-algebra$
53/46 Mathlib/RingTheory/AdjoinRoot.lean,Mathlib/RingTheory/Extension/Cotangent/Basic.lean,Mathlib/RingTheory/FiniteType.lean 3 1 ['github-actions'] nobody
20-25442
20 days ago
20-27065
20 days ago
20-27060
20 days
27042 Ruben-VandeVelde
author:Ruben-VandeVelde
feat: some WithZero lemmas Co-authored-by: matthewjasper <20113453+matthewjasper@users.noreply.github.com> Co-authored-by: Salvatore Mercuri --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) FLT t-algebra
label:t-algebra$
54/1 Mathlib/Algebra/Order/GroupWithZero/Canonical.lean 1 1 ['github-actions'] nobody
20-7623
20 days ago
20-7632
20 days ago
20-7677
20 days
26580 vasnesterov
author:vasnesterov
feat(Tactic/Order): translate linear orders to `Int` It was [pointed out](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/tactic.20for.20partial.20orders/near/515897754) that `order` is not complete for linear orders with lattice operations (while it remains complete for linear orders without lattice operations and for general lattices without assuming linearity). The problem for linear orders with lattice operations is NP-hard, but it can be translated from an arbitrary type to `Int` and then solved using a smart and efficient procedure (such as `omega`). This PR implements such a translation within the `order` tactic. Co-authored-by: Aaron Liu --- - [x] depends on: #26354 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-meta 302/22 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Order.lean,Mathlib/Tactic/Order/Graph/Basic.lean,Mathlib/Tactic/Order/Preprocessing.lean,Mathlib/Tactic/Order/ToInt.lean,MathlibTest/order.lean 7 4 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'vasnesterov'] nobody
19-30686
19 days ago
19-42594
19 days ago
19-44293
19 days
27049 BoltonBailey
author:BoltonBailey
doc(Analysis/BoxIntegral/Partition/Filter): field docstrings Split of #25917. Adds docstrings to the fields of this structure (Taken from the docstring of the structure itself). Note: this documentation was originally changed by asking Cursor (Claude 3.5 sonnet) to write the docstrings, but I think ultimately the docstring of the struct was reworked. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis 13/14 Mathlib/Analysis/BoxIntegral/Partition/Filter.lean 1 2 ['BoltonBailey', 'github-actions'] nobody
18-80500
18 days ago
19-82992
19 days ago
19-83212
19 days
26968 vihdzp
author:vihdzp
feat(Order/Concept): sets in a concept are codisjoint ...and other small lemmata. --- - [x] depends on: #26976 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order 33/2 Mathlib/Order/Concept.lean 1 8 ['github-actions', 'leanprover-community-bot-assistant', 'linesthatinterlace', 'mathlib4-dependent-issues-bot', 'plp127', 'vihdzp'] nobody
18-78208
18 days ago
18-78224
18 days ago
19-21376
19 days
27110 pechersky
author:pechersky
chore(Valued/WithVal): apply_symm_equiv valuation on the WIthVal is equal to the underlying valuation and simp tag --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-topology t-number-theory easy
label:t-algebra$
4/0 Mathlib/Topology/Algebra/Valued/WithVal.lean 1 1 ['github-actions'] nobody
18-62952
18 days ago
18-62955
18 days ago
18-63009
18 days
25814 vlad902
author:vlad902
feat(SimpleGraph): Weaker condition for paths in acyclic graphs `IsAcyclic.isPath_iff_chain'` defines a weaker condition for proving that a walk is a path, in particular it shows that rather than proving that all vertices in the support of a walk are distinct, one must only show that consecutive edges are distinct (e.g. every other vertex must be distinct.) This leads to a simple corollary that trails are also paths in acyclic graphs. I had a need for this when formalizing Cayley graphs, since this condition maps cleanly onto words in free groups being reduced. --- *This PR continues the work from #25630.* *Original PR: https://github.com/leanprover-community/mathlib4/pull/25630* t-combinatorics 43/0 Mathlib/Combinatorics/SimpleGraph/Acyclic.lean,Mathlib/Combinatorics/SimpleGraph/Paths.lean 2 2 ['github-actions', 'vlad902'] nobody
18-56580
18 days ago
50-26508
1 month ago
50-26490
50 days
26955 mariainesdff
author:mariainesdff
feat(LinearAlgebra/OnSup): extend linear maps to sums of modules Let `A` be a ring, `X, Y` be `A`-modules, and `M, N` be `A`-submodules of `X`. Given two linear maps `f : M →ₗ[A] Y` and `g : N →ₗ[A] Y` that agree on `M ∩ N`, there is a unique linear map `M + N →ₗ[A] Y` that simultaneously extends `f` and `g`. Co-authored-by: @AntoineChambert-Loir --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
153/0 Mathlib.lean,Mathlib/LinearAlgebra/OnSup.lean 2 15 ['AntoineChambert-Loir', 'eric-wieser', 'github-actions', 'wwylele'] nobody
18-36963
18 days ago
18-37030
18 days ago
19-1537
19 days
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/) t-algebra
label:t-algebra$
62/1 Mathlib/RingTheory/PowerSeries/Basic.lean,Mathlib/RingTheory/PowerSeries/Substitution.lean 2 5 ['Ruben-VandeVelde', 'github-actions', 'mariainesdff'] nobody
18-33841
18 days ago
22-39463
22 days ago
22-39513
22 days
27059 Komyyy
author:Komyyy
feat: Linear upper or lower sets topologies are completely normal The primary motivation for this theorem is to prove that Sierpiński space is completely normal. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology 77/1 Mathlib.lean,Mathlib/Topology/Order/UpperLowerSetTopology.lean,Mathlib/Topology/Separation/LinearUpperLowerSetTopology.lean 3 1 ['github-actions'] nobody
18-29832
18 days ago
19-54257
19 days ago
19-54240
19 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/) t-meta 18/22 Mathlib/Tactic/NormNum/Core.lean,Mathlib/Tactic/NormNum/Result.lean,Mathlib/Tactic/ReduceModChar.lean 3 2 ['eric-wieser', 'github-actions'] nobody
18-24140
18 days ago
21-22367
21 days ago
21-22350
21 days
27108 pechersky
author:pechersky
chore(RingTheory/AdicValuation): golf using WithZero.log with helper lemma of how `log` preserves order --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-number-theory
label:t-algebra$
15/16 Mathlib/Algebra/Order/GroupWithZero/Canonical.lean,Mathlib/RingTheory/DedekindDomain/AdicValuation.lean 2 2 ['YaelDillies', 'github-actions'] nobody
18-23556
18 days ago
18-23556
18 days ago
18-33347
18 days
27113 pechersky
author:pechersky
feat(RingTheory/SimpleRing/Principal): a commutative simple ring is a PID via `IsField` and new `IsField.isDomain` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
41/2 Mathlib.lean,Mathlib/Algebra/Field/IsField.lean,Mathlib/RingTheory/PrincipalIdealDomain.lean,Mathlib/RingTheory/SimpleRing/Principal.lean 4 4 ['alreadydone', 'github-actions'] nobody
18-19898
18 days ago
18-61302
18 days ago
18-61296
18 days
26282 AntoineChambert-Loir
author:AntoineChambert-Loir
feat: a theorem of Jordan on primitive subgroups of the permutation group A theorem of Jordan on the primitive subgroups of a permutation group: * if it contains a swap, it is equal to the permutation group, * if it contains a 3-cycle, it contains the alternating group. This PR continues the work from #24131. - [x] depends on: #26281 - [x] depends on: #26280 - [x] depends on: #26279 Original PR: https://github.com/leanprover-community/mathlib4/pull/24131 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import 1084/183 Mathlib.lean,Mathlib/Data/Set/Card.lean,Mathlib/GroupTheory/GroupAction/Jordan.lean,Mathlib/GroupTheory/GroupAction/MultiplePrimitivity.lean,Mathlib/GroupTheory/GroupAction/MultipleTransitivity.lean,Mathlib/GroupTheory/GroupAction/Primitive.lean,Mathlib/GroupTheory/GroupAction/SubMulAction/OfFixingSubgroup.lean,Mathlib/GroupTheory/GroupAction/SubMulAction/OfStabilizer.lean,Mathlib/GroupTheory/Perm/Cycle/Type.lean,Mathlib/SetTheory/Cardinal/Embedding.lean 10 n/a ['AntoineChambert-Loir', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'tb65536'] nobody
18-18963
18 days ago
unknown
unknown
27118 Timeroot
author:Timeroot
feat(Matrix/Charpoly/Eigs): Roots of Matrix.charpoly are the eigenvalues. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-algebra
label:t-algebra$
58/0 Mathlib/LinearAlgebra/Matrix/Charpoly/Eigs.lean,scripts/noshake.json 2 1 ['github-actions'] nobody
18-16356
18 days ago
18-55857
18 days ago
18-55900
18 days
22771 alreadydone
author:alreadydone
feat(Homotopy/Lifting): monodromy of covering maps and lifting criterion Definition 2.1 in https://ncatlab.org/nlab/show/monodromy. Also: + Extract `FundamentalGroupoid.map (f : C(X, Y)) : FundamentalGroupoid X ⥤ FundamentalGroupoid Y` from `fundamentalGroupoidFunctor : TopCat ⥤ CategoryTheory.Grpd` + Define `FundamentalGroup.map (f : C(X, Y)) (x : X) : FundamentalGroup X x →* FundamentalGroup Y (f x)` and `mapOfEq : FundamentalGroup X x →* FundamentalGroup Y y` that takes an assumption `f x = y`. + Redefine `FundamentalGroup` to be `End` rather than `Aut`: since `FundamentalGroupoid` is a groupoid, `End` already has a group structure. + Golf within the file FundamentalGroupoid/Basic. + Generalize `toArrow` up to `fromPath` in `FundamentalGroupoid/FundamentalGroup` from `X : TopCat` to `[TopologicalSpace X]`. Also golfs some proofs and redefines --- - [x] depends on: #22649 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology 193/147 Mathlib/AlgebraicTopology/FundamentalGroupoid/Basic.lean,Mathlib/AlgebraicTopology/FundamentalGroupoid/FundamentalGroup.lean,Mathlib/AlgebraicTopology/FundamentalGroupoid/InducedMaps.lean,Mathlib/AlgebraicTopology/FundamentalGroupoid/SimplyConnected.lean,Mathlib/CategoryTheory/Groupoid.lean,Mathlib/Topology/Covering.lean,Mathlib/Topology/Homotopy/HomotopyGroup.lean,Mathlib/Topology/Homotopy/Lifting.lean,Mathlib/Topology/Homotopy/Product.lean 9 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] PatrickMassot
assignee:PatrickMassot
17-40371
17 days ago
27-6762
27 days ago
134-72690
134 days
11563 YaelDillies
author:YaelDillies
feat: `∑ i ∈ s with hi : p i, f i hi` syntax for big operators Define new notation for `Finset.sum`/`Finset.prod`. `∑ i ∈ s with hi : p i, f i hi` now is notation for `∑ i : s.filter p, f i.1 (mem_filter.1 i.2).2`. --- - [x] depends on: #6795 Other notations we could have are * `∑ hi : i ∈ s, f i hi` as notation for `∑ i : s, f i.1 i.2` * `∑ hi : i ∈ s with p i, f i hi` as notation for `∑ i : s.filter p, f i.1 (mem_filter.1 i.2).1` * `∑ hi : i ∈ s with hpi : p i, f i hi hpi` as notation for `∑ i : s.filter p, f i.1 (mem_filter.1 i.2).1 (mem_filter.1 i.2).2` but Eric seems mildly unhappy about them. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-meta
label:t-algebra$
27/18 Mathlib/Algebra/BigOperators/Group/Finset/Defs.lean 1 28 ['YaelDillies', 'b-mehta', 'eric-wieser', 'github-actions', 'kbuzzard', 'kmill', 'leanprover-community-bot-assistant', 'leanprover-community-mathlib4-bot'] kmill
assignee:kmill
17-20047
17 days ago
17-20071
17 days ago
179-8027
179 days
25042 alreadydone
author:alreadydone
feat(Topology): restriction/extension of Trivialization and composition with Homeomorph --- - [x] depends on: #25041 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology 148/2 Mathlib/Topology/FiberBundle/Trivialization.lean,Mathlib/Topology/Maps/Basic.lean 2 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
17-19565
17 days ago
17-39763
17 days ago
73-23030
73 days
27072 eric-wieser
author:eric-wieser
feat(Data/Matrix): more lemmas about `Matrix.vecMulVec` Inspired by [#new members > Is this a reasonable formalization? @ 💬](https://leanprover.zulipchat.com/#narrow/channel/113489-new-members/topic/Is.20this.20a.20reasonable.20formalization.3F/near/528412531). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data 66/0 Mathlib/Data/Matrix/ConjTranspose.lean,Mathlib/Data/Matrix/Mul.lean 2 1 ['github-actions'] nobody
16-79620
16 days ago
19-27761
19 days ago
19-27802
19 days
27159 Parcly-Taxel
author:Parcly-Taxel
feat: IMO 1997 Q3 IMO 129/0 Archive.lean,Archive/Imo/Imo1997Q3.lean 2 5 ['Parcly-Taxel', 'eric-wieser', 'github-actions'] nobody
16-69387
16 days ago
17-30082
17 days ago
17-30070
17 days
25770 Parcly-Taxel
author:Parcly-Taxel
chore: fix more induction/recursor branch names These were found using the regex `\| h. =>` and `def.*rec.*\(h. :`. tech debt 134/115 Mathlib/Analysis/Convolution.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/Data/Fin/Tuple/Basic.lean,Mathlib/Data/Fin/Tuple/NatAntidiagonal.lean,Mathlib/Data/Nat/Factorization/Induction.lean,Mathlib/Data/Seq/Computation.lean,Mathlib/Data/Set/Card.lean,Mathlib/Data/WSeq/Basic.lean,Mathlib/FieldTheory/KummerExtension.lean,Mathlib/Logic/Function/Iterate.lean,Mathlib/NumberTheory/ArithmeticFunction.lean,Mathlib/NumberTheory/SumFourSquares.lean,Mathlib/NumberTheory/SumTwoSquares.lean,Mathlib/Order/SuccPred/Archimedean.lean,Mathlib/Order/Synonym.lean 15 11 ['Parcly-Taxel', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant'] nobody
16-69283
16 days ago
25-73346
25 days ago
48-55733
48 days
27200 rotarc75
author:rotarc75
feat(RingTheory/Ideal): oka predicates over ideals This PR introduces the notion of Oka predicates over the ideals of a ring. We usually speak of [Oka families](https://stacks.math.columbia.edu/tag/05K9) but predicates seemed more in line with mathlib's conventions. Currently this notions isn't used anywhere but we plan to make an other PR that proves that is all prime ideals of a ring are finitely generated, then this ring is Noetherian. We can also use Oka predicates to simplify the existing proof of [`IsPrincipalIdealRing.of_prime`](https://leanprover-community.github.io/mathlib4_docs/Mathlib/RingTheory/PrincipalIdealDomainOfPrime.html#IsPrincipalIdealRing.of_prime). Co-authored-by: Anthony Fernandes --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra
label:t-algebra$
53/0 Mathlib.lean,Mathlib/RingTheory/Ideal/Oka.lean 2 1 ['github-actions'] nobody
16-38859
16 days ago
16-38859
16 days ago
16-39758
16 days
27207 pechersky
author:pechersky
feat(Topology/WithVal): ValuativeRel (WithVal v) with a helper valuation defined that does not pierce defeq --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-topology
label:t-algebra$
23/0 Mathlib/Topology/Algebra/Valued/WithVal.lean 1 1 ['github-actions'] nobody
16-28781
16 days ago
16-28782
16 days ago
16-29096
16 days
27210 YaelDillies
author:YaelDillies
feat: `MonoidHom.toHomUnits` is a monoid hom From Toric --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) toric large-import t-algebra
label:t-algebra$
21/4 Mathlib/Algebra/Group/Units/Hom.lean 1 1 ['github-actions'] nobody
16-27368
16 days ago
16-27719
16 days ago
16-27862
16 days
27182 eric-wieser
author:eric-wieser
feat: add bundled versions of `Equiv.cast` These are essentially the non-categorical versions of `eqToHom`. These are helpful to state some functorial results about things like `DFinsupp.equivCongrLeft` (with the alternative being to use an evil triangle somewhere instead). [#Is there code for X? > LinearEquiv.cast / AddEquiv.cast etc @ 💬](https://leanprover.zulipchat.com/#narrow/channel/217875-Is-there-code-for-X.3F/topic/LinearEquiv.2Ecast.20.2F.20AddEquiv.2Ecast.20etc/near/521390380) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
31/0 Mathlib/Algebra/Algebra/Equiv.lean,Mathlib/Algebra/Group/Equiv/Defs.lean,Mathlib/Algebra/Module/Equiv/Defs.lean,Mathlib/Algebra/Ring/Equiv.lean 4 3 ['github-actions', 'pechersky', 'plp127'] nobody
16-17547
16 days ago
16-82510
16 days ago
16-82552
16 days
27226 xcloudyunx
author:xcloudyunx
feat(Combinatorics/SimpleGraph): Add Subgraph.inclusion_edge_apply_coe and inclusion_edgeSet_apply_coe This PR continues the work from #25248. Original PR: https://github.com/leanprover-community/mathlib4/pull/25248 new-contributor t-combinatorics 14/0 Mathlib/Combinatorics/SimpleGraph/Subgraph.lean 1 1 ['github-actions'] nobody
15-72397
15 days ago
15-73816
15 days ago
15-73872
15 days
27014 yuanyi-350
author:yuanyi-350
feat(GroupTheory/Perm/Fin): add Fin.cycleIcc and refactor cycleRange In this PR, I define the permutation `cycleIcc i j hij`, which is the cycle `(i i+1 .... j)` leaving `(0 ... i-1)` and `(j+1 ... n-1)` unchanged. In other words, it rotates elements in `[i, j]` one step to the right. Also I prove some properties of `cycleIcc i j hij` such as the fact that it is a cycle and its cycleType is `j - i`. **This definition is used to prove the following result:** ``` theorem succAbove_comp_cycleIcc [NeZero n] (x : Fin (n + 1) → L) (i j : Fin (n + 1)) (eq : x i = x j) (lt : i < j) x ∘ i.succAbove = x ∘ j.succAbove ∘ (cycleIcc hij) ``` More clearly, `x ∘ i.succAbove` and `x ∘ j.succAbove` are `Fin n → L` types. For example, when `n = 6, i = 2, j = 5` and `x i = x j` ``` x ∘ i.succAbove = (x 0, x 1, x 3, x 4, x 5, x 6) x ∘ j.succAbove = (x 0, x 1, x 2, x 3, x 4, x 6) ``` We have ``` (x 0, x 1, x 3, x 4, x 5, x 6) --(cycleIcc)--->(x 0, x 1, x 5, x 3, x 4, x 6) = (x 0, x 1, x 2, x 3, x 4, x 6) ``` --- Migrated from #24139 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
216/26 Mathlib/Algebra/Group/Fin/Basic.lean,Mathlib/Data/Fin/Basic.lean,Mathlib/Data/Fin/Embedding.lean,Mathlib/Data/Fin/SuccPred.lean,Mathlib/GroupTheory/Perm/Fin.lean 5 55 ['faenuccio', 'github-actions', 'mbkybky', 'yuanyi-350'] faenuccio
assignee:faenuccio
15-61032
15 days ago
17-33113
17 days ago
20-25864
20 days
26870 grunweg
author:grunweg
feat: mdifferentiableOn_section_of_mem_baseSet₀ From the path towards geodesics and the Levi-Civita connection. Co-authored-by: Patrick Massot --- - [x] depends on: #26866 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-differential-geometry 125/0 Mathlib/Geometry/Manifold/VectorBundle/MDifferentiable.lean 1 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
15-29538
15 days ago
15-29700
15 days ago
15-29861
15 days
27021 grunweg
author:grunweg
feat: custom elaborators for differential geometry Add two sets of custom elaborators for differential geometry, to - infer the model with corners in `MDifferentiable{WithinAt,At,On}` or `ContMDiff{WithinAt,At,On}` expressions from the local context, and provide shorter notation in that setting - do the same for mfderiv: `mfderiv% f` is shorthand for `mfderiv I J f`; `mfderiv[s] f x` is short for `mfderivWithin I J f s` - convert a fibre bundle section from a dependent section to a function into the total space, making working with differentiability of sections of fibre bundles less cumbersome This was [discussed on zulip](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Differential.20geometry.20elaborators.20experiment/with/528035295), to overall broad consensus. This code has substantial tests and has been tried in the branch in #26221 (uncovering minor issues, but not substantial ones). The implementation itself is of prototype quality and will be cleaned up in the future. Once it is more robust, more differential geometry files can be converted to use it. Co-authored-by: Patrick Massot ----------- I agree that merging not fully polished code is not ideal, but propose doing so for two reasons: - the work in #26221 used these elaborators extensively (to test them). Reverting those changes, merging the code, only to re-apply them is not a good use of time. Merging this PR now enables merging the work in #26221 soon. - the feature is clearly useful and not going away: in the files that use it, it works well already. Holding off on further adopting, but merging it now seems like a good compromise. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-differential-geometry t-meta 782/0 Mathlib.lean,Mathlib/Geometry/Manifold/Elaborators.lean,Mathlib/Geometry/Manifold/Traces.lean,MathlibTest/DifferentialGeometry/Elaborators.lean,scripts/noshake.json 5 4 ['github-actions', 'grunweg', 'sgouezel'] nobody
15-24647
15 days ago
20-47576
20 days ago
20-47649
20 days
27179 euprunin
author:euprunin
chore: golf `sub_convs_eq` using `field_simp` and `grind` t-algebra
label:t-algebra$
2/10 Mathlib/Algebra/ContinuedFractions/Computation/Approximations.lean 1 4 ['euprunin', 'github-actions', 'grunweg'] nobody
15-7579
15 days ago
17-2504
17 days ago
17-2548
17 days
22782 alreadydone
author:alreadydone
feat(Topology): étalé space associated to a predicate on sections --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology 886/160 Mathlib.lean,Mathlib/AlgebraicGeometry/ProjectiveSpectrum/StructureSheaf.lean,Mathlib/Data/Set/Operations.lean,Mathlib/Geometry/Manifold/Sheaf/Smooth.lean,Mathlib/Logic/Equiv/Basic.lean,Mathlib/Topology/EtaleSpace.lean,Mathlib/Topology/IsLocalHomeomorph.lean,Mathlib/Topology/Sheaves/LocalPredicate.lean,Mathlib/Topology/Sheaves/Sheafify.lean,Mathlib/Topology/Sheaves/Stalks.lean 10 12 ['AntoineChambert-Loir', 'alreadydone', 'github-actions', 'jcommelin', 'leanprover-community-bot-assistant'] nobody
14-77891
14 days ago
25-81680
25 days ago
25-82396
25 days
26667 mariainesdff
author:mariainesdff
feat(FieldTheory/SplittingField/IsSplittingField): add IsScalarTower.splits, IsScalarTower.isAlgebraic Co-authored-by: @faenuccio --- - [ ] depends on: #26666 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
29/0 Mathlib/Algebra/Polynomial/Lifts.lean,Mathlib/FieldTheory/SplittingField/IsSplittingField.lean 2 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'tb65536'] nobody
14-74765
14 days ago
17-27233
17 days ago
17-27839
17 days
23940 YaelDillies
author:YaelDillies
feat: polytopes From Toric Co-authored-by: Matthew Johnson --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) toric t-analysis 65/0 Mathlib.lean,Mathlib/Geometry/Convex/Polytope.lean,Mathlib/Geometry/Convex/README.md 3 9 ['Parcly-Taxel', 'YaelDillies', 'eric-wieser', 'github-actions', 'jsm28', 'leanprover-community-bot-assistant'] nobody
14-53261
14 days ago
51-7806
1 month ago
111-79927
111 days
26074 oliver-butterley
author:oliver-butterley
feat(Mathlib.Dynamics.BirkhoffSum): add 2 lemmas for birkhoffSum/birkhoffAverage concerning ae_eq observables If two observables are `ae_eq` then the birkhoffSum/birkhoffAverage of those observables are `ae_eq`. Motivation: - Generally it is useful to be able to swap to observables which are `ae_eq`. - Specifically this is useful to prove Birkhoff's pointwise ergodic theorem by first proving the result for integrable and measurable observables and then using this to deduce the result with just the requirement of integrable. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-dynamics 44/0 Mathlib.lean,Mathlib/Dynamics/BirkhoffSum/QuasiMeasurePreserving.lean 2 10 ['github-actions', 'oliver-butterley', 'sgouezel'] nobody
14-43794
14 days ago
14-43812
14 days ago
44-46662
44 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/) t-algebra
label:t-algebra$
141/26 Mathlib.lean,Mathlib/Data/Quot.lean,Mathlib/Data/Setoid/Basic.lean,Mathlib/GroupTheory/Congruence/Defs.lean,Mathlib/GroupTheory/Congruence/GroupWithZero.lean 5 22 ['ADedecker', 'eric-wieser', 'github-actions'] nobody
14-29562
14 days ago
16-46348
16 days ago
16-56792
16 days
27245 rirarika
author:rirarika
MvPolynomial.Irreducible --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra
label:t-algebra$
88/0 Mathlib.lean,Mathlib/Algebra/MvPolynomial/Irreducible.lean 2 3 ['alreadydone', 'github-actions', 'mbkybky'] nobody
14-22675
14 days ago
14-49164
14 days ago
14-49207
14 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 337/0 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/NormNum/NormNumI.lean,MathlibTest/norm_numI.lean 4 35 ['Whysoserioushah', 'eric-wieser', 'github-actions', 'hrmacbeth'] nobody
14-8565
14 days ago
15-12043
15 days ago
15-16360
15 days
27261 Sebi-Kumar
author:Sebi-Kumar
feat(Topology): add definition for subpaths Define subpaths as restrictions of paths to subintervals, reparameterized to have domain `[0, 1]` and possibly with a reverse of direction. Prove their basic properties. This serves as an alternative to `Path.truncate` which is useful for the explicit construction of certain homotopies, in particular regarding the concatenation of subpaths. --- To provide additional context, this is my first time contributing to Mathlib, and I am doing so as a part of the Fields Undergraduate Summer Research Program hosted at Western University. My intention for this file is for it to be used when proving that the fundamental group of the sphere is trivial (following the proof from Hatcher's "Algebraic Topology"). [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-topology 148/0 Mathlib.lean,Mathlib/Topology/Subpath.lean 2 1 ['github-actions'] nobody
14-1698
14 days ago
14-12329
14 days ago
14-12376
14 days
27264 pechersky
author:pechersky
feat(Topology/ValuedField): range of valuation on competion is the same as base field and other helper API to prepare for ValuativeTopology --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology 60/0 Mathlib/Topology/Algebra/Valued/ValuedField.lean 1 1 ['github-actions'] nobody
14-547
14 days ago
14-557
14 days ago
14-601
14 days
27265 pechersky
author:pechersky
feat(Topology/Valued): discrete topology on a valued field when trivial valuation or when there is a nonzero term in the valuation codomain that is smaller than all nonzero valuations --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology 33/0 Mathlib/Topology/Algebra/Valued/ValuationTopology.lean 1 1 ['github-actions'] nobody
14-543
14 days ago
14-547
14 days ago
14-590
14 days
25833 loefflerd
author:loefflerd
feat(Counterexamples): topologists' sine curve Define the "topologists' sine curve" in R^2, and show that its closure is connected but not path-connected. This formalization is part of the bachelor thesis of Daniele Bolla at UniDistance Switzerland. Co-authored-by: Daniele Bolla [daniele.bolla@stu.fernuni.ch](mailto:daniele.bolla@stu.fernuni.ch) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) migrated-from-branch t-topology 219/1 Counterexamples.lean,Counterexamples/TopologistsSineCurve.lean,Mathlib/Topology/Connected/PathConnected.lean 3 13 ['Ruben-VandeVelde', 'github-actions', 'loefflerd', 'sgouezel'] nobody
13-85378
13 days ago
13-85511
13 days ago
49-33268
49 days
26484 peabrainiac
author:peabrainiac
feat(Geometry/Diffeology): basics of diffeological spaces Introduces diffeological spaces, smooth maps between them, the D-topology and the standard diffeology on finite-dimensional normed spaces. --- This PR continues the work from #21969. t-differential-geometry 471/0 Mathlib.lean,Mathlib/Geometry/Diffeology/Basic.lean,docs/references.bib 3 9 ['JovanGerb', 'github-actions', 'lecopivo', 'peabrainiac'] nobody
13-69847
13 days ago
34-67165
1 month ago
34-71916
34 days
25920 BoltonBailey
author:BoltonBailey
feat(Data/Finsupp/Basic): `Finsupp.optionElim'` Similar to how Finsupp.cons constructs a map Fin (n + 1) →₀ M from a map Fin n →₀ M, we define Finsupp.optionElim' to construct a map Option α →₀ M from a map α →₀ M, given an additional value for none. We base this on the new optionEquiv definition. As a function, it behaves as Option.elim', hence the name. We prove a variety of API lemmas, based on those for Finsupp.cons, to bring the definitions more in line with the contents of Data/Finsupp/Fin. We also refactor to a new file to help avoid a too-long file and make this more analogous to Finsupp.cons Original PR: https://github.com/leanprover-community/mathlib4/pull/13861 - [x] depends on: #26309 migrated-from-branch t-data 124/25 Mathlib/Algebra/Category/MonCat/Adjunctions.lean,Mathlib/Data/Finsupp/Option.lean 2 13 ['BoltonBailey', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
13-67312
13 days ago
13-67332
13 days ago
35-74315
35 days
26371 Timeroot
author:Timeroot
feat(NumberTheory): Niven's theorem This file proves Niven's theorem, that the only rational cosines of angles that are rational multiples of pi, are [-1, -1/2, 0, 1/2, 1]. This is one of the theorems missing from 1000.yaml. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-number-theory 119/0 Mathlib.lean,Mathlib/NumberTheory/Niven.lean,docs/1000.yaml 3 9 ['Timeroot', 'github-actions', 'grunweg', 'plp127'] nobody
13-29555
13 days ago
38-8941
1 month ago
38-8987
38 days
26880 agjftucker
author:agjftucker
feat(Calculus/FDeriv/Partial): `hasStrictFDerivAt_uncurry_coprod` concerning partial derivatives Confident that other contributions will follow (e.g. #26300), I begin this file with only the result needed to apply the implicit function theorem to a curried function. --- - [x] depends on: #26742 [This dependency is very slight.] [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor 126/0 Mathlib.lean,Mathlib/Analysis/Calculus/FDeriv/Partial.lean 2 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
13-5557
13 days ago
13-5557
13 days ago
16-83137
16 days
27242 hugh-fox
author:hugh-fox
feat: add Gauss-like formula for sums of digit sums Adds `sum_digit_sum_base_pow_eq` to show a Gauss-like formula across sums of digit sums. This relies on an additional two simp lemmas, named `digits_sum_eq_self`, `digits_sum_base_mul_cancel`. Lastly, includes a specialization (which is a good bit simpler than the general formula) to base 10 named `sum_digit_sum_ten_pow_eq`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-data new-contributor 113/0 Mathlib/Data/Nat/Digits/Lemmas.lean 1 5 ['github-actions', 'hugh-fox', 'kckennylau'] nobody
13-4460
13 days ago
14-68238
14 days ago
14-68284
14 days
27216 D-Thomine
author:D-Thomine
feat(Cardinal/Finite): ENat powers and cardinality This PR continues the work from #25574. Original PR: https://github.com/leanprover-community/mathlib4/pull/25574 t-algebra
label:t-algebra$
204/5 Mathlib.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/Data/ENat/Pow.lean,Mathlib/SetTheory/Cardinal/Finite.lean 4 12 ['D-Thomine', 'eric-wieser', 'github-actions'] nobody
12-31364
12 days ago
13-34276
13 days ago
14-51347
14 days
27312 pechersky
author:pechersky
feat(RingTheory/Valuation): the trivial valuation, as One (Valuation R Γ₀) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-number-theory
label:t-algebra$
54/0 Mathlib/Algebra/GroupWithZero/Hom.lean,Mathlib/RingTheory/Valuation/Basic.lean 2 1 ['github-actions'] nobody
12-6469
12 days ago
12-6531
12 days ago
12-6523
12 days
24530 chrisflav
author:chrisflav
feat(RingTheory): faithfully flat ring maps Co-authored by: Joël Riou --- - [x] depends on: #24375 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
89/1 Mathlib.lean,Mathlib/Algebra/Ring/Equiv.lean,Mathlib/RingTheory/RingHom/FaithfullyFlat.lean,Mathlib/RingTheory/RingHom/Flat.lean 4 7 ['chrisflav', 'erdOne', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
11-58852
11 days ago
12-30024
12 days ago
68-10000
68 days
26035 fbarroero
author:fbarroero
feat(Analysis/Polynomial/MahlerMeasure): the Mahler measure of a complex polynomial We introduce the Mahler measure of a complex polynomial and prove some basic facts. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis 127/1 Mathlib.lean,Mathlib/Analysis/Polynomial/MahlerMeasure.lean,Mathlib/MeasureTheory/Integral/CircleIntegral.lean 3 1 ['github-actions'] nobody
11-15528
11 days ago
44-18684
1 month ago
44-18687
44 days
27082 staroperator
author:staroperator
feat(Order/WellFoundedSet): add `Set.IsPWO.exists_le_minimal`, `Set.IsPWO.exists_minimal`, `Set.IsPWO.exists_minimalFor` which are the `IsPWO` version of `exists_minimal_le_of_wellFoundedLT` and others. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-order 22/0 Mathlib/Order/WellFoundedSet.lean 1 4 ['alreadydone', 'github-actions', 'staroperator'] nobody
10-67169
10 days ago
19-16583
19 days ago
19-16628
19 days
27357 jcreedcmu
author:jcreedcmu
feat(Algebra/Module/Submodule): add `submoduleMap` for isometries Per [discussion on Zulip](https://leanprover.zulipchat.com/#narrow/channel/217875-Is-there-code-for-X.3F/topic/Analog.20of.20LinearEquiv.2EsubmoduleMap.20for.20AffineIsometryEquiv.3F), add a version of `.submoduleMap` for `LinearIsometry` and `LinearIsometryEquiv` by analogy with `LinearMap.submoduleMap` and `LinearEquiv.submoduleMap`. --- new-contributor t-algebra
label:t-algebra$
56/0 Mathlib.lean,Mathlib/Analysis/Normed/Operator/LinearIsometrySubmoduleMap.lean 2 12 ['Ruben-VandeVelde', 'eric-wieser', 'github-actions', 'jcreedcmu'] nobody
9-84952
9 days ago
10-3735
10 days ago
10-3786
10 days
27370 euprunin
author:euprunin
chore(Tactic/CancelDenoms): golf `cancel_factors_eq` t-meta 1/11 Mathlib/Tactic/CancelDenoms/Core.lean 1 1 ['github-actions'] nobody
9-80773
9 days ago
9-80792
9 days ago
9-80840
9 days
26448 YaelDillies
author:YaelDillies
refactor: simplify `(f₁ ⊗ₘ f₂) ≫ (g₁ ⊗ₘ g₂)` to `(f₁ ≫ g₁) ⊗ₘ (f₂ ≫ g₂)` ... instead of the other way around. This is motivated by the fact that homs happening "in parallel" is a non-concept (time along a branch can always be reparametrised), while homs happening "in series" is a well-defined concept. One should not simp the well-defined concept into the non-concept but instead the other way around. This is also motivated by the advent of the `mon_tauto` simp set in #26057. From Toric --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) toric t-category-theory 115/119 Mathlib/Algebra/Category/ModuleCat/Monoidal/Basic.lean,Mathlib/Algebra/Category/ModuleCat/Presheaf/Monoidal.lean,Mathlib/CategoryTheory/Bicategory/End.lean,Mathlib/CategoryTheory/Dialectica/Monoidal.lean,Mathlib/CategoryTheory/Enriched/Basic.lean,Mathlib/CategoryTheory/Enriched/FunctorCategory.lean,Mathlib/CategoryTheory/GradedObject/Braiding.lean,Mathlib/CategoryTheory/GradedObject/Monoidal.lean,Mathlib/CategoryTheory/Localization/Monoidal.lean,Mathlib/CategoryTheory/Monoidal/Braided/Basic.lean,Mathlib/CategoryTheory/Monoidal/Braided/Reflection.lean,Mathlib/CategoryTheory/Monoidal/Cartesian/Basic.lean,Mathlib/CategoryTheory/Monoidal/Category.lean,Mathlib/CategoryTheory/Monoidal/Free/Basic.lean,Mathlib/CategoryTheory/Monoidal/Functor.lean,Mathlib/CategoryTheory/Monoidal/FunctorCategory.lean,Mathlib/CategoryTheory/Monoidal/Internal/Limits.lean,Mathlib/CategoryTheory/Monoidal/Limits.lean,Mathlib/CategoryTheory/Monoidal/Mon_.lean,Mathlib/CategoryTheory/Monoidal/NaturalTransformation.lean,Mathlib/CategoryTheory/Monoidal/Opposite.lean,Mathlib/CategoryTheory/Monoidal/Preadditive.lean,Mathlib/CategoryTheory/Monoidal/Transport.lean,Mathlib/CategoryTheory/Monoidal/Types/Coyoneda.lean 24 13 ['YaelDillies', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'robin-carlier', 'yuma-mizuno'] nobody
9-51853
9 days ago
9-51872
9 days ago
33-29598
33 days
27174 ADedecker
author:ADedecker
chore(OreLocalization): generalize some results from rings to monoids with zeros --- My motivation is getting a more conceptual construction of [ValuativeRel.ValueGroupWithZero](https://leanprover-community.github.io/mathlib4_docs/Mathlib/RingTheory/Valuation/ValuativeRel.html#ValuativeRel.ValueGroupWithZero), but I think this is of independent interest. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
104/73 Mathlib.lean,Mathlib/RingTheory/OreLocalization/Basic.lean,Mathlib/RingTheory/OreLocalization/NonZeroDivisors.lean,Mathlib/RingTheory/OreLocalization/Ring.lean 4 2 ['github-actions', 'leanprover-community-bot-assistant'] nobody
9-47126
9 days ago
9-47583
9 days ago
16-76153
16 days
27040 Scarlett-le
author:Scarlett-le
feat(Geometry/Euclidean/Sphere/Power): add power of a point theorems Add the definition of power of a point and fundamental theorems relating point positions to intersection distances: * `Sphere.power`: The power of a point with respect to a sphere, defined as the square of the distance from the point to the center minus the square of the radius. * `Sphere.power_eq_zero_iff_mem_sphere`: A point lies on the sphere if and only if its power is zero. * `Sphere.power_pos_iff_dist_center_gt_radius`: The power is positive if and only if the point is outside the sphere. * `Sphere.power_neg_iff_dist_center_lt_radius`: The power is negative if and only if the point is inside the sphere. * `Sphere.mul_dist_eq_power_of_dist_center_gt_radius`: For external points, the product of intersection distances equals the power. * `Sphere.mul_dist_eq_neg_power_of_dist_center_lt_radius`: For internal points, the product equals the negative power. * `Sphere.mul_dist_eq_abs_power`: General form relating intersection distance products to absolute power. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-euclidean-geometry 138/1 Mathlib/Geometry/Euclidean/Sphere/Power.lean 1 3 ['alreadydone', 'github-actions'] jsm28
assignee:jsm28
9-42756
9 days ago
20-10223
20 days ago
20-10763
20 days
26847 joelriou
author:joelriou
feat: multicoequalizers in the category of types This PR gives a concrete criteria for a multicofork in the category of types to be a multicoequalizer, and this is used in order to show that if a (sub)set `A : Set X` is the union of certain subsets `U i`, then the type `A` is the multicoequalizer of the `U i`s along their intersections `V i j`. (A similar result for `Subpresheaf` rather than `Set` will be deduced in a separate PR, and this shall be very important in the study of the homotopy theory of simplicial sets, as this will allow the construction of morphisms from horns.) --- - [x] depends on: #25823 - [x] depends on: #22205 - [x] depends on: #26037 This PR continues the work from #23872. Original PR: https://github.com/leanprover-community/mathlib4/pull/23872 t-category-theory 96/0 Mathlib.lean,Mathlib/CategoryTheory/Limits/Types/Multicoequalizer.lean 2 n/a ['adomani', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
9-35864
9 days ago
unknown
unknown
27277 artie2000
author:artie2000
feat(Logic/Equiv): `Equiv` on `Subtype` implies equivalence of existence statements * Add lemmas stating that an `Equiv` between `Subtypes` implies the equivalence of the corresponding `Exists` and `ExistsUnique` propositions. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data 9/0 Mathlib/Logic/Equiv/Defs.lean 1 6 ['YaelDillies', 'artie2000', 'eric-wieser', 'github-actions'] nobody
8-83038
8 days ago
13-66472
13 days ago
13-68691
13 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/) t-order 394/0 Mathlib.lean,Mathlib/Order/SigmaCompleteLattice.lean 2 3 ['PierreQuinton', 'github-actions', 'vihdzp'] nobody
8-39683
8 days ago
8-51221
8 days ago
8-51268
8 days
27424 vihdzp
author:vihdzp
feat: interval in archimedean field contains fraction with large enough denominator This is a slight generalization of `exists_rat_btwn` that can be used, for instance, to prove that there's a dyadic rational between any two elements. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) maintainer-merge t-algebra
label:t-algebra$
13/11 Mathlib/Algebra/Order/Archimedean/Basic.lean 1 2 ['Ruben-VandeVelde', 'github-actions'] nobody
8-7942
8 days ago
8-7942
8 days ago
8-41104
8 days
27427 alreadydone
author:alreadydone
chore(RingTheory): use `extend` instead of `abbrev` in `IsS(emis)impleModule` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
46/37 Mathlib/Algebra/Category/ModuleCat/Simple.lean,Mathlib/Algebra/Module/PID.lean,Mathlib/LinearAlgebra/RootSystem/Irreducible.lean,Mathlib/LinearAlgebra/Semisimple.lean,Mathlib/RepresentationTheory/Maschke.lean,Mathlib/RingTheory/Length.lean,Mathlib/RingTheory/SimpleModule/Basic.lean,Mathlib/RingTheory/SimpleModule/Rank.lean 8 4 ['alreadydone', 'github-actions', 'leanprover-bot'] nobody
8-7930
8 days ago
8-7930
8 days ago
8-7913
8 days
27107 AntoineChambert-Loir
author:AntoineChambert-Loir
feat(GroupTheory/GroupAction/SubMulAction/Combination) : combinations and group actions `Nat.Combination X n` is the type all `s : Finset X` such that `s.card = n`. This PR provides some API for this subtype and the `SubMulAction` it inherits when a group acts on `X`. It will be used in conjunction with the description of some maximal subgroups of `Equiv.Perm X` to construct primitive actions. Question on the names: when `X` is a fintype, there is docs#Finset.powersetCard` that gives the same object, as a docs#Finset. But the present PR also applies when `X` is infinite. Then maybe `Nat.Combination` should be renamed as `Set.powersetCard`? --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
318/0 Mathlib.lean,Mathlib/Data/Nat/Choose/Basic.lean,Mathlib/GroupTheory/GroupAction/SubMulAction/Combination.lean 3 2 ['github-actions', 'tb65536'] nobody
8-2559
8 days ago
18-72460
18 days ago
18-72504
18 days
26783 matthewjasper
author:matthewjasper
feat(RingTheory/Flat): Add theorems relating Submodule.torsion and Module.Flat Co-authored-by: Kevin Buzzard --- This PR continues the work from #25334. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) FLT new-contributor t-algebra
label:t-algebra$
205/0 Mathlib.lean,Mathlib/Algebra/Algebra/Bilinear.lean,Mathlib/Algebra/Module/LocalizedModule/Basic.lean,Mathlib/RingTheory/Flat/TorsionFree.lean,Mathlib/RingTheory/Ideal/IsPrincipal.lean 5 1 ['github-actions'] nobody
8-1531
8 days ago
27-33973
27 days ago
27-34001
27 days
27453 pechersky
author:pechersky
feat(Topology/UniformSpace/Ultra): completion is ultra uniformity iff base is Supersedes #24628 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology 159/5 Mathlib.lean,Mathlib/Order/Filter/NAry.lean,Mathlib/Order/Filter/Prod.lean,Mathlib/Topology/Constructions/SumProd.lean,Mathlib/Topology/UniformSpace/Defs.lean,Mathlib/Topology/UniformSpace/Ultra/Basic.lean,Mathlib/Topology/UniformSpace/Ultra/Completion.lean 7 1 ['github-actions'] nobody
7-74462
7 days ago
7-74522
7 days ago
7-74516
7 days
27455 pechersky
author:pechersky
chore(NumberTheory/Padics/Hensel): rephrase using `aeval` This is easier to use at call site, because on need not pass `Polynomial.map (algebraMap _ _ )` in the use of `hensels_lemma` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) tech debt t-algebra t-number-theory
label:t-algebra$
157/138 Mathlib/NumberTheory/Padics/Hensel.lean 1 1 ['github-actions'] nobody
7-68304
7 days ago
7-68359
7 days ago
7-68356
7 days
27460 IvanRenison
author:IvanRenison
feat(Combinatorics/SimpleGraph/Walk): add theorems about membership on the support of `Walk.concat` This contribution was created as part of the Utrecht Summerschool "Formalizing Mathematics in Lean" in July 2025. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics 18/0 Mathlib/Combinatorics/SimpleGraph/Walk.lean 1 1 ['github-actions'] nobody
7-30481
7 days ago
7-42082
7 days ago
7-42123
7 days
27464 IvanRenison
author:IvanRenison
feat(Combinatorics/SimpleGraph/Paths): add lemma `SimpleGraph.Walk.IsPath.ne_of_mem_support_of_append` This contribution was created as part of the Utrecht Summerschool "Formalizing Mathematics in Lean" in July 2025. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics 7/0 Mathlib/Combinatorics/SimpleGraph/Paths.lean 1 1 ['github-actions'] nobody
7-30465
7 days ago
7-39797
7 days ago
7-39846
7 days
27468 IvanRenison
author:IvanRenison
feat(Combinatorics/SimpleGraph): add theorem `SimpleGraph.Connected.diff_dist_adj` This contribution was created as part of the Utrecht Summerschool "Formalizing Mathematics in Lean" in July 2025. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics 16/0 Mathlib/Combinatorics/SimpleGraph/Metric.lean 1 1 ['github-actions'] nobody
7-30459
7 days ago
7-31980
7 days ago
7-32078
7 days
24192 alreadydone
author:alreadydone
feat(RingTheory): semisimple Wedderburn–Artin existence --- - [x] depends on: #24119 - [x] depends on: #23963 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
469/67 Mathlib/Algebra/Algebra/Pi.lean,Mathlib/Algebra/Ring/Equiv.lean,Mathlib/LinearAlgebra/DFinsupp.lean,Mathlib/Order/CompleteSublattice.lean,Mathlib/RingTheory/SimpleModule/Basic.lean,Mathlib/RingTheory/SimpleModule/IsAlgClosed.lean,Mathlib/RingTheory/SimpleModule/Isotypic.lean,Mathlib/RingTheory/SimpleModule/WedderburnArtin.lean,docs/1000.yaml 9 5 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
7-29763
7 days ago
7-29912
7 days ago
75-74852
75 days
27472 guelmi94
author:guelmi94
feat(Combinatorics/SimpleGraph/Walk): add lemma `support_injective` This contribution was created as part of the Utrecht Summerschool "Formalizing Mathematics in Lean" in July 2025. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-combinatorics 3/0 Mathlib/Combinatorics/SimpleGraph/Walk.lean 1 1 ['github-actions'] nobody
7-25313
7 days ago
7-25316
7 days ago
7-25364
7 days
26679 robin-carlier
author:robin-carlier
feat(CategoryTheory/Limits/Shapes/Pullback/Categorical): 2-functoriality of `CatCommSqOver` This PR uses the notion of categorical cospan transforms from #26412 and its bicategory-like notations from #26447 to provide API for 2-functoriality of the construction `CatCommSqOver F G X`. We show that `ψ : CatCospanTransform F G F' G'` defines a functor `CatCommSqOver F G X ⥤ CatCommSqOver F' G' X`, and that a functor `U : X ⥤ Y` induces a functor `CatCommSqOver F G Y ⥤ CatCommSqOver F G X` via precomposition. We give the battery of lemma that shows that these constructions are components of a `Cat`-valued "bipseudofunctor", although we cannot state it this way to keep things unbundled and universe polymorphic. --- - [x] depends on: #26447 I apologize in advance, for this one is very boring. As usual, the higher order lemmas are found by aesop_cat and are not marked simp, but I still want to state these explicitly so that in case automation goes wrong, "manual formal bicategory manipulations" remain an option. A design choice was made here. Instead of stating this kind of functoriality for the categorical pullback itself, I chose to state everything in terms of `CatCommSqOver`, i.e in terms of the pseudofunctorial construction corepresented by the categorical pullback. The rationale here is that while we could have done everything only at the level of the categorical pullback itself, I believe this design will allow for easier manipulations of categorical pullback *squares*. Actual bifunctoriality of the categorical pullback (and thus equivalence invariance, which is the key point of the notion compared to the strict pullback) will be in future PRs. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory 364/1 Mathlib/CategoryTheory/Limits/Shapes/Pullback/Categorical/Basic.lean 1 4 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'robin-carlier'] nobody
7-24340
7 days ago
7-24340
7 days ago
16-57981
16 days
27447 eric-wieser
author:eric-wieser
refactor: rename `Rel` to `Set.Rel`, restore the old `Rel` Many users are confused that Rel no longer means what it used to. Since the design is not obvious, let's put it in a namespace that makes the choice obvious. This then restores the old definition of `Rel`, as an abbrev; it's conceivable that many users were just using this as a shorthand, and this stops them being broken by #25587. Such users will of course be broken if they used [the old API](https://github.com/leanprover-community/mathlib4/blob/59bd63c72671849996d64c5d3b5f24a36333483c%5E/Mathlib/Data/Rel.lean). This way, users bumping from 4.21.0 to 4.22.0 and using `Rel` only as a shorthand will not be broken. [#mathlib4 > Changing `Rel` to `Set (α × β)`, to help uniform spaces @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Changing.20.60Rel.60.20to.20.60Set.20.28.CE.B1.20.C3.97.20.CE.B2.29.60.2C.20to.20help.20uniform.20spaces/near/528531852) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order 134/116 Mathlib/CategoryTheory/Category/RelCat.lean,Mathlib/Combinatorics/Hall/Basic.lean,Mathlib/Combinatorics/SimpleGraph/Basic.lean,Mathlib/Combinatorics/SimpleGraph/Subgraph.lean,Mathlib/Data/PFun.lean,Mathlib/Data/Rel.lean,Mathlib/Order/Filter/Partial.lean,Mathlib/Order/KrullDimension.lean,Mathlib/Order/Rel/GaloisConnection.lean,Mathlib/Order/RelSeries.lean,Mathlib/RingTheory/Length.lean,Mathlib/Topology/Partial.lean,Mathlib/Topology/UniformSpace/Basic.lean 13 3 ['YaelDillies', 'eric-wieser', 'github-actions'] nobody
7-24300
7 days ago
7-40432
7 days ago
7-80784
7 days
25951 themathqueen
author:themathqueen
feat(Analysis/InnerProductSpace/MulOpposite): defines the inner product on opposite spaces This pr defines the inner product on opposite spaces. - [x] depends on: #25949 Motivation for having the inner product structure on the opposite: One application comes up in non-commutative graphs, which are defined on a finite-dimensional C*-algebra with a faithful and positive functional (a Hilbert space structure can be induced by the defined faithful and positive functional (will be added to a pr soon)). For example, we'd need the Hilbert space structure to be defined on the opposite space to define the isomorphism: `(A →ₗ[ℂ] B) ≃ₗ[ℂ] TensorProduct ℂ B Aᵐᵒᵖ`, where `A`, `B` are again finite-dimensional C*-algebras with faithful and positive functionals. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor 71/0 Mathlib.lean,Mathlib/Analysis/InnerProductSpace/MulOpposite.lean 2 6 ['github-actions', 'j-loreaux', 'mathlib4-dependent-issues-bot', 'themathqueen'] nobody
7-18798
7 days ago
9-36206
9 days ago
26-57717
26 days
27441 judithludwig
author:judithludwig
feat(RingTheory/Polynomial/Quotient): Lemma on PIDs This is part of a course project at Heidelberg University: https://matematiflo.github.io/CompAssistedMath2025/ feat(RingTheory/Polynomial/Quotient): add lemma: Let $$R$$ be an integral domain and assume $$R[X]$$ is a PID, then $$R$$ is a field. This lemma is useful for proving that some rings are not PIDs, such as $$\mathbb{Z}[X]$$. Co-authored-by: Philipp Sivov @Silipp182 Co-authored-by: Veliyan Taslev @hubavelko --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
11/0 Mathlib/RingTheory/Polynomial/Quotient.lean 1 3 ['alreadydone', 'github-actions'] nobody
7-15056
7 days ago
8-6042
8 days ago
8-6087
8 days
26912 pechersky
author:pechersky
chore(Algebra/Ring/Subring): simp tag `Subring.smul_def` s-multiplying by a subtype is easiest to manipulate when both terms are in the ambient type. Many places that had to use the _def lemma for a rewrite, or to include it in a simp set, no longer have to. Ported from #25308 --- [![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. maintainer-merge t-algebra
label:t-algebra$
68/67 Mathlib/Algebra/Algebra/Subalgebra/Basic.lean,Mathlib/Algebra/Field/Subfield/Basic.lean,Mathlib/Algebra/Group/Subgroup/Actions.lean,Mathlib/Algebra/Group/Submonoid/MulAction.lean,Mathlib/Algebra/Module/LocalizedModule/Basic.lean,Mathlib/Algebra/Module/LocalizedModule/Exact.lean,Mathlib/Algebra/Module/LocalizedModule/IsLocalization.lean,Mathlib/Algebra/Module/LocalizedModule/Submodule.lean,Mathlib/Algebra/Ring/Periodic.lean,Mathlib/Algebra/Ring/Subring/Basic.lean,Mathlib/Algebra/Ring/Subsemiring/Basic.lean,Mathlib/Analysis/CStarAlgebra/Basic.lean,Mathlib/FieldTheory/KummerExtension.lean,Mathlib/GroupTheory/GroupAction/Defs.lean,Mathlib/GroupTheory/GroupAction/MultiplePrimitivity.lean,Mathlib/GroupTheory/GroupAction/MultipleTransitivity.lean,Mathlib/GroupTheory/GroupAction/SubMulAction/OfFixingSubgroup.lean,Mathlib/GroupTheory/GroupAction/SubMulAction/OfStabilizer.lean,Mathlib/LinearAlgebra/RootSystem/Irreducible.lean,Mathlib/LinearAlgebra/RootSystem/RootPositive.lean,Mathlib/LinearAlgebra/RootSystem/WeylGroup.lean,Mathlib/RingTheory/Etale/Kaehler.lean,Mathlib/RingTheory/LocalProperties/Projective.lean,Mathlib/RingTheory/Localization/InvSubmonoid.lean,Mathlib/RingTheory/OreLocalization/Basic.lean 25 16 ['eric-wieser', 'github-actions', 'j-loreaux', 'linesthatinterlace', 'pechersky'] nobody
7-9712
7 days ago
10-2602
10 days ago
21-17476
21 days
26299 adomani
author:adomani
perf: the `commandStart` linter only acts on modified files Introduces an `IO.Ref` to allow the `commandStart` linter to only run on files that git considers modified with respect to `master`. The linter is also active on files that have had some error, as these are likely being modified! The PR should also mitigate the speed-up that the linter introduced: [#mathlib4 > A whitespace linter @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/A.20whitespace.20linter/near/525091877) Assuming that this goes well, a similar mechanism could be applied to several linters that do not need to run on all code, just on the modified code. Implementation detail: the linter is currently either on or off in "whole" files. It may be also a future development to make this more granular and only run the linter on "modifed commands in modified files", but this is not currently the plan for this modification! --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-linter 48/0 Mathlib/Tactic/Linter/CommandStart.lean 1 5 ['adomani', 'github-actions', 'grunweg', 'leanprover-bot'] nobody
6-83001
6 days ago
39-28185
1 month ago
39-32816
39 days
27152 xroblot
author:xroblot
feat(RingTheory/Ideal): prove transitivity for the relative norm --- - [x] depends on: #26070 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
150/13 Mathlib/Algebra/Algebra/Tower.lean,Mathlib/RingTheory/Ideal/Norm/RelNorm.lean,Mathlib/RingTheory/Ideal/Prime.lean,Mathlib/RingTheory/IntegralClosure/IntegralRestrict.lean,Mathlib/RingTheory/Localization/AtPrime.lean,Mathlib/RingTheory/Localization/FractionRing.lean 6 5 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'riccardobrasca', 'xroblot'] riccardobrasca
assignee:riccardobrasca
6-79696
6 days ago
16-81398
16 days ago
17-5946
17 days
25182 YaelDillies
author:YaelDillies
feat: `(M →* N₁) ≃* (M →* N₂)` if `N₁ ≃* N₂` The names were discussed on [Zulip](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Naming.20congruence.20of.20maps) but no consensus was reached due to lack of engagement. The names I choose here are consistent with [`ContinuousLinearEquiv.continuousAlternatingMapCongrLeft`](https://leanprover-community.github.io/mathlib4_docs/find/?pattern=ContinuousLinearEquiv.continuousAlternatingMapCongrLeft#doc) and around. From Toric --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) toric t-algebra
label:t-algebra$
116/18 Mathlib/Algebra/Category/Grp/ForgetCorepresentable.lean,Mathlib/Algebra/Category/Grp/LargeColimits.lean,Mathlib/Algebra/Category/MonCat/ForgetCorepresentable.lean,Mathlib/Algebra/Group/Equiv/Basic.lean,Mathlib/GroupTheory/FiniteAbelian/Duality.lean 5 20 ['YaelDillies', 'b-mehta', 'eric-wieser', 'github-actions'] eric-wieser
assignee:eric-wieser
6-50563
6 days ago
8-19780
8 days ago
66-11040
66 days
27497 ScottCarnahan
author:ScottCarnahan
feat(RingTheory/PowerSeries/Binomial): add basic lemmas, golf This PR adds two simp lemmas for binomial power series, and generalizes the hypotheses of `binomialSeries_nat`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
17/19 Mathlib/RingTheory/PowerSeries/Binomial.lean 1 3 ['ScottCarnahan', 'github-actions', 'wwylele'] nobody
6-39697
6 days ago
6-76502
6 days ago
6-76496
6 days
27498 Komyyy
author:Komyyy
feat: Group isomorphisms between (`Equiv.Perm`|`alternatingGroup`)s Required to prove that A_n is simple iff n = 3 or 5 ≤ n(#26051). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
29/0 Mathlib/Algebra/Group/End.lean,Mathlib/GroupTheory/SpecificGroups/Alternating.lean 2 1 ['github-actions'] nobody
6-16792
6 days ago
6-75947
6 days ago
6-75931
6 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/) t-topology 21/0 Mathlib/Topology/UnitInterval.lean 1 1 ['github-actions'] nobody
6-12248
6 days ago
6-16327
6 days ago
6-16371
6 days
27515 gaetanserre
author:gaetanserre
feat: `ProbabilityTheory.cdf_eq_real` for measure on `unitInterval` Given a probability measure `μ` on `I`, the CDF of the pushforward of `μ` along `Subtype.val` is equal to the measure of the closed interval. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-measure-probability 9/0 Mathlib/Probability/CDF.lean 1 1 ['github-actions'] nobody
6-12225
6 days ago
6-17891
6 days ago
6-17935
6 days
27517 gaetanserre
author:gaetanserre
feat: a `MeasurableEmbedding` has a measurable left inverse Definition of the measurable left inverse of a `MeasurableEmbedding`. Co-authored-by: Rémy Degenne --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-measure-probability 29/0 Mathlib/MeasureTheory/MeasurableSpace/Embedding.lean 1 1 ['github-actions'] nobody
6-12031
6 days ago
6-15652
6 days ago
6-15696
6 days
26350 mans0954
author:mans0954
feature(RingTheory/RootsOfUnity/Basic) : rootsOfUnity coercions This PR continues the work from #25215. Original PR: https://github.com/leanprover-community/mathlib4/pull/25215 t-algebra
label:t-algebra$
22/0 Mathlib/RingTheory/RootsOfUnity/Basic.lean 1 2 ['github-actions', 'mans0954'] nobody
6-8019
6 days ago
38-50304
1 month ago
38-50345
38 days
25905 mans0954
author:mans0954
feat(RingTheory/Polynomial/SmallDegreeVieta): polynomial versions of results in Algebra.QuadraticDiscriminant This PR continues the work from #25605. Original PR: https://github.com/leanprover-community/mathlib4/pull/25605 t-algebra
label:t-algebra$
73/8 Mathlib/RingTheory/Polynomial/SmallDegreeVieta.lean 1 31 ['github-actions', 'kckennylau', 'mans0954'] nobody
6-7936
6 days ago
47-33824
1 month ago
47-33867
47 days
27437 kckennylau
author:kckennylau
feat(RingTheory/Valuation): some lemmas about comparing with 1 and 0 and with each other *From the 2025 Local Class Field Theory Workshop.* --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
109/22 Mathlib/NumberTheory/Padics/ValuativeRel.lean,Mathlib/RingTheory/Valuation/Basic.lean,Mathlib/RingTheory/Valuation/Extension.lean,Mathlib/RingTheory/Valuation/ValuativeRel.lean 4 18 ['erdOne', 'github-actions', 'kckennylau', 'matthewjasper', 'pechersky'] nobody
6-6358
6 days ago
8-18682
8 days ago
8-18723
8 days
27361 101damnations
author:101damnations
feat(Algebra/Homology/AlternatingConst): generalize to any appropriate complex shape and pair of maps Given an object `X : C` and endomorphisms `φ, ψ : X ⟶ X` such that `φ ∘ ψ = ψ ∘ φ = 0`, this PR defines the periodic chain and cochain complexes `... ⟶ X --φ--> X --ψ--> X --φ--> X --ψ--> 0` and `0 ⟶ X --ψ--> X --φ--> X --ψ--> X --φ--> ...` (or more generally for any complex shape `c` on `ℕ` where `c.Rel i j` implies `i` and `j` have different parity). We calculate the homology of these periodic complexes. This generalizes some of the current content of the file, which works for the chain complex where `ψ = 0` and `φ = Id`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) maintainer-merge t-algebra
label:t-algebra$
129/13 Mathlib/Algebra/Homology/AlternatingConst.lean 1 3 ['github-actions', 'kbuzzard'] nobody
6-2198
6 days ago
6-2198
6 days ago
9-85111
9 days
27527 peabrainiac
author:peabrainiac
feat(Topology): some `IsOpenMap` lemmas Some lemmas for `IsOpenMap` that I needed. I've also added variants for `IsClosedMap` to maintain symmetry in the API. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology 46/0 Mathlib/Topology/Constructions.lean 1 2 ['github-actions', 'peabrainiac'] nobody
5-76861
5 days ago
5-77399
5 days ago
5-77421
5 days
26478 JovanGerb
author:JovanGerb
chore(LibraryRewrite): replace `rw??` with `rw?` As suggested by @YaelDillies, now `rw?` overwrites Lean core's implementation of `rw?`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta 56/49 Mathlib/Tactic/Widget/LibraryRewrite.lean,MathlibTest/LibraryRewrite.lean,MathlibTest/rewrites.lean 3 5 ['YaelDillies', 'erdOne', 'github-actions', 'leanprover-community-bot-assistant'] nobody
5-72086
5 days ago
5-82464
5 days ago
20-57810
20 days
27500 Komyyy
author:Komyyy
feat: the Riemann zeta function is meromorphic Also proves that the Hurwitz zeta function is meromorphic. This PR is split from #27499 to leave a good git diff history. --- The `large-import` change occurs only in the new module, so it poses no problem. - [x] depends on: #27499 This PR continues the work from #25597. Original PR: https://github.com/leanprover-community/mathlib4/pull/25597 large-import t-analysis 51/3 Mathlib.lean,Mathlib/Analysis/Meromorphic/Complex.lean,Mathlib/Analysis/Meromorphic/Gamma.lean 3 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
5-65404
5 days ago
5-66220
5 days ago
5-66835
5 days
27536 joelriou
author:joelriou
feat(Algebra/Homology): complementary embeddings Given two embeddings `e₁ : c₁.Embedding c` and `e₂ : c₂.Embedding c` of complex shapes, we introduce a property `e₁.AreComplementary e₂` saying that the image subsets of the indices of `c₁` and `c₂` form a partition of the indices of `c`. If `e₁.IsTruncLE` and `e₂.IsTruncGE`, and `K : HomologicalComplex C c`, we construct a quasi-isomorphism `shortComplexTruncLEX₃ToTruncGE` between the cokernel of `K.ιTruncLE e₁ : K.truncLE e₁ ⟶ K` and `K.truncGE e₂`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-category-theory
label:t-algebra$
327/0 Mathlib.lean,Mathlib/Algebra/Homology/Embedding/AreComplementary.lean 2 1 ['github-actions'] nobody
5-41956
5 days ago
5-41962
5 days ago
5-42007
5 days
27504 joelriou
author:joelriou
feat(CategoryTheory/Limits): filtered colimits of types In this file, given a functor `F : J ⥤ Type w₀` from a filtered category `J`, we compute the equivalence relation generated by `F.ColimitTypeRel` on `(j : J) × (F.obj j)`. Given `c : CoconeTypes F`, we deduce a lemma `Functor.CoconeTypes.injective_descColimitType_iff_of_isFiltered` which gives a concrete condition under which the map `F.descColimitType c : F.ColimitType → c.pt` is injective, which is an important step when proving `c.IsColimit`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory 134/0 Mathlib.lean,Mathlib/CategoryTheory/Limits/Types/ColimitType.lean,Mathlib/CategoryTheory/Limits/Types/ColimitTypeFiltered.lean 3 5 ['Ruben-VandeVelde', 'github-actions', 'joelriou'] nobody
5-40221
5 days ago
5-49765
5 days ago
5-56618
5 days
27537 vasnesterov
author:vasnesterov
feat(Analysis): radius of convergence for binomial series Introduce the binomial series as `FormalMultilinearSeries`, and prove that its radius of convergence is `1`. --- - [x] depends on: #22518 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) This PR continues the work from #22538. Original PR: https://github.com/leanprover-community/mathlib4/pull/22538 t-analysis 83/0 Mathlib.lean,Mathlib/Analysis/Analytic/Binomial.lean,Mathlib/RingTheory/Binomial.lean 3 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
5-35579
5 days ago
5-36976
5 days ago
5-37027
5 days
26270 vasnesterov
author:vasnesterov
chore(Analysis/Analytic): split `Analytic.Basic` Move the results on the radius of convergence from `Analytic/Basic.lean` to a new file `Analytic/ConvergenceRadius.lean`. --- - [x] depends on: #26255 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) tech debt t-analysis 450/431 Mathlib.lean,Mathlib/Analysis/Analytic/Basic.lean,Mathlib/Analysis/Analytic/ConvergenceRadius.lean,Mathlib/Analysis/Analytic/OfScalars.lean,Mathlib/Analysis/Analytic/RadiusLiminf.lean 5 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
5-35334
5 days ago
5-35334
5 days ago
6-25073
6 days
27482 alreadydone
author:alreadydone
chore(RingTheory/SimpleModule): golf and generalize lifting_property --- Build succeeded but there's a strange post-build step error. https://github.com/leanprover-community/mathlib4/actions/runs/16527173966/job/46744293147?pr=27482 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
11/14 Mathlib/RingTheory/SimpleModule/Basic.lean,Mathlib/RingTheory/SimpleModule/InjectiveProjective.lean 2 2 ['github-actions', 'smorel394'] nobody
5-34161
5 days ago
7-17971
7 days ago
7-17955
7 days
27548 euprunin
author:euprunin
chore(Control/Functor/Multivariate): remove use of `erw` in `f` (`private def f`) t-data 1/1 Mathlib/Control/Functor/Multivariate.lean 1 1 ['github-actions'] nobody
5-23030
5 days ago
5-23036
5 days ago
5-23087
5 days
27550 chrisflav
author:chrisflav
chore(RingTheory/Polynomial): add `ker_constantCoeff` and `constantCoeff_surjective` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
9/0 Mathlib/Algebra/Polynomial/Coeff.lean,Mathlib/RingTheory/Polynomial/Ideal.lean 2 1 ['github-actions'] nobody
5-21831
5 days ago
5-21902
5 days ago
5-21885
5 days
26798 robin-carlier
author:robin-carlier
feat(CategoryTheory/Monoidal/DayConvolution): `LawfulDayConvolutionMonoidalCategoryStruct` Given monoidal categories `C`, `V` and a category `D` with a pre-existing `MonoidalCategoryStruct`, we introduce a typeclass `LawfulDayConvolutionMonoidalCategoryStruct C V D` that bundles the required data and equations that the structure on `D` must have to be a monoidal subcategory of `C ⥤ V` if the latter was endowed with the day convolution monoidal structure. The data in question is that of a faithful functor `ι : D ⥤ C ⥤ V`, as well as explicit natural transformations `ι.obj d ⊠ (ι.obj d') ⟶ tensor C ⋙ ι.obj (d ⊗ d')` that exhibit `ι.obj (d ⊗ d')` as a Day convolution of `ι.obj d` and `(ι.obj d')`, as well as similar data asserting that `ι.obj (𝟙_ D)` is a Day convolution unit. The equations required are identical to the ones that characterize the unitors and associators for Day convolution with respect to the Kan extensions units. Given such a structure, using that the corresponding relations hold in `C ⥤ V`, we show that the monoidal category structure on `D` defines a `MonoidalCategory D`, i.e that all the required equations such as the pentagon/triangular equalities, bifunctoriality of the tensor product etc. are satisfied. Thus, we can think of `LawfulDayConvolutionMonoidalCategoryStruct C V D` as a constructor for monoidal categories. While this is a step towards a Day convolution monoidal structure in (a type alias) `C ⥤ V`, the framework is yet incomplete, as it assumes a pre-existing monoidal category structure. We will give constructors for (`MonoidalCategoryStruct` and) `LawfulDayConvolutionMonoidalCategoryStruct C V D` with various degree of definitional control over the resulting structure in a forthcoming PR. --- - [x] depends on: #25757 I recommend the reviewer to at least have a glance at #26820 to see where this is going, and how this one fits in the design I have in mind. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory 336/8 Mathlib/CategoryTheory/Monoidal/DayConvolution.lean 1 4 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
5-21312
5 days ago
5-21335
5 days ago
18-83812
18 days
27554 euprunin
author:euprunin
chore(LinearAlgebra/PiTensorProduct): `grind` away use of `erw` in `lifts_zero` t-algebra
label:t-algebra$
1/1 Mathlib/LinearAlgebra/PiTensorProduct.lean 1 1 ['github-actions'] nobody
5-16468
5 days ago
5-16479
5 days ago
5-16523
5 days
26031 joelriou
author:joelriou
feat(Algebra/Homology): the derived category of a linear abelian category is linear --- - [x] depends on: #25931 This PR continues the work from #24596. Original PR: https://github.com/leanprover-community/mathlib4/pull/24596 t-category-theory 71/0 Mathlib.lean,Mathlib/Algebra/Homology/DerivedCategory/Linear.lean,Mathlib/Algebra/Homology/HomotopyCategory/Shift.lean,Mathlib/Algebra/Homology/HomotopyCategory/SingleFunctors.lean 4 n/a ['AntoineChambert-Loir', 'github-actions', 'joelriou', 'mathlib4-dependent-issues-bot'] nobody
5-9073
5 days ago
unknown
unknown
27566 wwylele
author:wwylele
feat(Data/Real): Archimedean.embedReal is a ring hom when M is an ordered ring Also shows that this ends up the same as `LinearOrderedField.inducedOrderRingHom` for fields --- This is a spin-off from #27268 ~~because I got bored~~ . This is not in a high priority as I don't need it for anything yet, but the last lemma shows that `embedReal` is a generalization of `LinearOrderedField.inducedOrderRingHom` (which is only stated for field, and I didn't find when I was making the group embedding). Perhaps we should refactor `Mathlib/Algebra/Order/CompleteField.lean` with the definition here. Indeed, if we replace every `ℝ` with `(R : Type*)[ConditionallyCompleteLinearOrderedField R]` in `Data/Real/Embedding.lean`, the proof still works. What do you think? [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-data 220/3 Mathlib/Data/Real/Embedding.lean 1 1 ['github-actions'] nobody
5-3001
5 days ago
5-3008
5 days ago
5-3060
5 days
27567 themathqueen
author:themathqueen
feat(LinearAlgebra/TensorProduct/Tower): add `lid` and `assoc` tensor lemmas This adds `TensorProduct.lid_tensor` and `TensorProduct.assoc_tensor`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
21/0 Mathlib/LinearAlgebra/TensorProduct/Tower.lean 1 2 ['github-actions', 'themathqueen'] nobody
5-1497
5 days ago
5-2289
5 days ago
5-2333
5 days
27288 themathqueen
author:themathqueen
feat(LinearAlgebra/TensorProduct/Basic): semi-linearize `map` and `lift` Semi-linearizing `TensorProduct.map`. Part of #27353. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
29/18 Mathlib/Algebra/Category/ModuleCat/ChangeOfRings.lean,Mathlib/LinearAlgebra/TensorProduct/Basic.lean,Mathlib/RingTheory/Coalgebra/Hom.lean 3 4 ['ADedecker', 'eric-wieser', 'github-actions', 'themathqueen'] nobody
5-297
5 days ago
5-297
5 days ago
8-24821
8 days
24015 alreadydone
author:alreadydone
feat(RingTheory): lemmas on finiteness of `LinearMap` and `Module.End` --- One less lemma than #24012, but with the advantage of not depending on #23963. - [x] depends on: #24115 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
137/81 Mathlib/Algebra/Module/LinearMap/End.lean,Mathlib/GroupTheory/GroupAction/SubMulAction.lean,Mathlib/LinearAlgebra/BilinearMap.lean,Mathlib/LinearAlgebra/Dual/Lemmas.lean,Mathlib/LinearAlgebra/Projection.lean,Mathlib/RingTheory/Finiteness/Basic.lean,Mathlib/RingTheory/SimpleModule/Basic.lean 7 22 ['alreadydone', 'erdOne', 'eric-wieser', 'github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'leanprover-community-mathlib4-bot', 'mathlib4-dependent-issues-bot'] erdOne
assignee:erdOne
4-81554
4 days ago
5-4944
5 days ago
107-81381
107 days
27544 eric-wieser
author:eric-wieser
feat: upgrade lflip to a `LinearEquiv` This deletes some `aux` definitions without deprecation. This is helpful for building the version of `DFinsupp.lsum` for bilinear maps. A handful of existing users of `lflip` now need to add an explicit `toLinearMap`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
24/35 Mathlib/LinearAlgebra/BilinearForm/Basic.lean,Mathlib/LinearAlgebra/BilinearMap.lean,Mathlib/LinearAlgebra/TensorPower/Basic.lean,Mathlib/LinearAlgebra/TensorProduct/Associator.lean,Mathlib/LinearAlgebra/TensorProduct/Graded/External.lean,Mathlib/LinearAlgebra/TensorProduct/Tower.lean,Mathlib/RingTheory/PiTensorProduct.lean,Mathlib/RingTheory/TensorProduct/Basic.lean 8 1 ['github-actions'] nobody
4-81084
4 days ago
4-81084
4 days ago
4-81426
4 days
27378 peakpoint
author:peakpoint
refactor(Geometry/Euclidean/Projection): redefine projection and reflection for affine subspaces This PR continues the work from #25578. Original PR: https://github.com/leanprover-community/mathlib4/pull/25578 new-contributor t-euclidean-geometry 316/317 Mathlib/Analysis/Normed/Affine/ContinuousAffineMap.lean,Mathlib/Analysis/Normed/Affine/Isometry.lean,Mathlib/Geometry/Euclidean/Circumcenter.lean,Mathlib/Geometry/Euclidean/Projection.lean 4 4 ['github-actions', 'leanprover-community-bot-assistant', 'peakpoint'] nobody
4-77832
4 days ago
4-78935
4 days ago
8-48270
8 days
27562 hrmacbeth
author:hrmacbeth
chore: deduplicate "transform at location" methods Many metaprograms have the following general structure: the input is an expression `e` and the output is a new expression `e'`, together with a proof that `e = e'`. Such a metaprogram produces a variety of tactics: it may be used to modify the goal, a specified hypothesis, or (via `Tactic.Location`) a combination of these. Roughly the same code for this is repeated throughout the library, for the tactics `ring_nf`, `abel_nf`, `norm_num`, `push_neg` and `reduce_mod_char`; possibly it originates from the `ring_nf` version, #552. This PR extracts this repeated code to a stand-alone function in `Mathlib.Util.AtLocation`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-meta 115/166 Mathlib.lean,Mathlib/Tactic/Abel.lean,Mathlib/Tactic/NormNum/Core.lean,Mathlib/Tactic/Push.lean,Mathlib/Tactic/ReduceModChar.lean,Mathlib/Tactic/Ring/RingNF.lean,Mathlib/Util/AtLocation.lean,MathlibTest/abel.lean,MathlibTest/norm_num.lean 9 4 ['github-actions', 'grunweg', 'hrmacbeth'] nobody
4-74731
4 days ago
4-74731
4 days ago
5-8339
5 days
25788 Parcly-Taxel
author:Parcly-Taxel
feat: number of edges in the Turán graph We provide two theorems, the first `card_edgeFinset_turanGraph` providing the exact number of edges and the other `card_edgeFinset_turanGraph_le` providing a (slightly) looser bound whose main advantage is its lack of integer division/modulus operations. The bound in `card_edgeFinset_turanGraph_le` is also the bound provided in [Motzkin and Straus (1965)](https://doi.org/10.4153%2FCJM-1965-053-6). large-import t-combinatorics 132/0 Mathlib/Combinatorics/SimpleGraph/Turan.lean,Mathlib/Data/Nat/ModEq.lean 2 3 ['YaelDillies', 'github-actions', 'leanprover-community-bot-assistant'] nobody
4-73043
4 days ago
4-73067
4 days ago
50-35348
50 days
27018 Komyyy
author:Komyyy
feat: Finite product of Alexandrov-discrete spaces is Alexandrov-discrete --- - [x] depends on: #27016 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology 93/9 Mathlib/Data/Set/Lattice.lean,Mathlib/Data/Set/Lattice/Image.lean,Mathlib/Order/Filter/Ker.lean,Mathlib/Topology/AlexandrovDiscrete.lean,Mathlib/Topology/NhdsKer.lean 5 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
4-51790
4 days ago
4-64777
4 days ago
4-64761
4 days
26225 Raph-DG
author:Raph-DG
feat(AlgebraicGeometry): Add some minimal API for orders on schemes In this PR we add some minimal api for the ordering on schemes defined in #26204. We chose split these PRs because we expect there will be more discussion about this API, and having the preorder instance is useful in its own right without much added API. - [] depends on: #26204 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebraic-geometry 14/0 Mathlib/AlgebraicGeometry/Properties.lean,Mathlib/AlgebraicGeometry/Scheme.lean 2 4 ['Raph-DG', 'github-actions', 'joelriou', 'leanprover-community-bot-assistant'] nobody
4-51585
4 days ago
4-51585
4 days ago
40-31232
40 days
24804 Moises-Herradon-Cueto
author:Moises-Herradon-Cueto
feat(CategoryTheory/Limits/Preserves/Shapes): show that if a functor preserves limits, so does `Over.post` If a functor `F` preserves limits (of a certain shape, finite, or of a certain size), then so does the induced functor on `Over` categories. From Toric Co-authored-by: Yaël Dillies --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) toric new-contributor t-category-theory 125/0 Mathlib.lean,Mathlib/CategoryTheory/Limits/Preserves/Shapes/Over.lean,Mathlib/CategoryTheory/WithTerminal/Basic.lean 3 17 ['Moises-Herradon-Cueto', 'YaelDillies', 'erdOne', 'github-actions', 'joelriou'] nobody
4-48809
4 days ago
66-24489
2 months ago
72-28882
72 days
27283 Louddy
author:Louddy
feat(SkewMonoidAlgebra): maps on/to SkewMonoidAlgebra Add the definition of many maps regarding skew monoid algebras and lemmas associated to them. These all have their analogues for `MonoidAlgebra`. Co-authored-by: María Inés de Frutos Fernández <[mariaines.dff@gmail.com](mailto:mariaines.dff@gmail.com)> --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-algebra
label:t-algebra$
237/0 Mathlib/Algebra/SkewMonoidAlgebra/Basic.lean 1 1 ['github-actions'] nobody
4-48670
4 days ago
13-51256
13 days ago
13-51305
13 days
27253 Louddy
author:Louddy
feat(SkewMonoidAlgebra): SkewMonoidAlgebra/Support Add lemmas regarding the support of a skew monoid algebra. It is currently missing a few lemmas compared to `MonoidAlgebra.support`. (See TODO.) These will be added as more results are available on `SkewMonoidAlgebra`. Co-authored-by: María Inés de Frutos Fernández <[mariaines.dff@gmail.com](mailto:mariaines.dff@gmail.com)> --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
100/0 Mathlib.lean,Mathlib/Algebra/SkewMonoidAlgebra/Support.lean 2 1 ['github-actions'] nobody
4-48648
4 days ago
14-27184
14 days ago
14-27196
14 days
25292 YaelDillies
author:YaelDillies
feat: the `ConvexCone` generated by a set Define `ConvexCone.copy` and `ConvexCone.hull` and use them to golf the `CompleteLattice` instance. From Toric --- - [x] depends on: #25291 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-convex-geometry toric 94/35 Mathlib/Analysis/Convex/Cone/Basic.lean,Mathlib/Geometry/Convex/Cone/Basic.lean 2 8 ['YaelDillies', 'b-mehta', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
4-45947
4 days ago
5-39859
5 days ago
42-78185
42 days
27582 IvanRenison
author:IvanRenison
feat(Combinatorics/SimpleGraph/Paths): add theorem `SimpleGraph.Walk.IsPath.isPath_concat` This contribution was created as part of the Utrecht Summerschool "Formalizing Mathematics in Lean" in July 2025. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics 7/0 Mathlib/Combinatorics/SimpleGraph/Paths.lean 1 1 ['github-actions'] nobody
4-44728
4 days ago
4-44754
4 days ago
4-44803
4 days
27583 RemyDegenne
author:RemyDegenne
feat: in a countable discrete measurable space, every measure is s-finite The instance is placed in the `WithDensity` file, because that's where we have the instance `SFinite (c • μ)` that I use in the proof. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-measure-probability 4/0 Mathlib/MeasureTheory/Measure/WithDensity.lean 1 1 ['github-actions'] nobody
4-44689
4 days ago
4-44692
4 days ago
4-44738
4 days
27581 eric-wieser
author:eric-wieser
fix(Data/BitVec): remove a `SMul` instance diamond When the `Nat`- and `Int`-action typeclasses and their instances were upstreamed, they changed to a different (and worse) defeq. This removes the mathlib instances and proves the old defeq still holds propositionally. Also move some theorems out of the `BitVec` file that are not about `BitVec` at all, and are about `Fin`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-data 57/54 Mathlib/Data/BitVec.lean,Mathlib/Data/ZMod/Defs.lean 2 2 ['eric-wieser', 'github-actions'] nobody
4-44219
4 days ago
4-46505
4 days ago
4-46556
4 days
27584 RemyDegenne
author:RemyDegenne
feat(Probability): lemmas about `Kernel.discard` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-measure-probability 22/1 Mathlib/MeasureTheory/Measure/GiryMonad.lean,Mathlib/Probability/Kernel/Basic.lean,Mathlib/Probability/Kernel/Composition/Comp.lean,Mathlib/Probability/Kernel/Composition/MeasureComp.lean 4 1 ['github-actions'] nobody
4-42928
4 days ago
4-42935
4 days ago
4-42983
4 days
27585 RemyDegenne
author:RemyDegenne
feat(Probability): `posterior_eq_withDensity_of_countable` This PR adds a simpler version of `posterior_eq_withDensity` for the case of a countable space. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-measure-probability 12/0 Mathlib/Probability/Kernel/Posterior.lean 1 1 ['github-actions'] nobody
4-42669
4 days ago
4-42681
4 days ago
4-42726
4 days
27586 RemyDegenne
author:RemyDegenne
feat(Probability): `Kernel.comp_const` `κ ∘ₖ Kernel.const α μ = Kernel.const α (κ ∘ₘ μ)` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-measure-probability 7/0 Mathlib/Probability/Kernel/Composition/MeasureComp.lean 1 1 ['github-actions'] nobody
4-42380
4 days ago
4-42392
4 days ago
4-42437
4 days
26016 CBirkbeck
author:CBirkbeck
Iterated derivatives of tsum's within some open set. We add some IteratedDerivWithin versions of deriv_tsum using the new SummableLocallyUniformly API. This PR continues the work from #25096. Original PR: https://github.com/leanprover-community/mathlib4/pull/25096 t-analysis 139/0 Mathlib.lean,Mathlib/Algebra/BigOperators/Pi.lean,Mathlib/Analysis/Calculus/IteratedDeriv/Lemmas.lean,Mathlib/Topology/Algebra/InfiniteSum/TsumUniformlyOn.lean,Mathlib/Topology/Algebra/InfiniteSum/UniformOn.lean 5 3 ['CBirkbeck', 'github-actions', 'leanprover-community-bot-assistant'] nobody
4-42307
4 days ago
4-46034
4 days ago
26-86348
26 days
27587 RemyDegenne
author:RemyDegenne
feat(Probability): instances for `Kernel` on empty types --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-measure-probability 20/0 Mathlib/Probability/Kernel/Basic.lean,Mathlib/Probability/Kernel/Defs.lean 2 1 ['github-actions'] nobody
4-40016
4 days ago
4-40022
4 days ago
4-40069
4 days
26660 strihanje01
author:strihanje01
feat(Combinatorics/Additive/VerySmallDoubling): weak non-commutative Kneser's theorem add theorem about the structure of a doubling smaller than the golden ratio --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import new-contributor t-combinatorics 859/5 Mathlib/Combinatorics/Additive/VerySmallDoubling.lean 1 61 ['YaelDillies', 'github-actions', 'strihanje01'] nobody
4-20772
4 days ago
21-9844
21 days ago
26-60063
26 days
27597 mitchell-horner
author:mitchell-horner
feat(Combinatorics/SimpleGraph): define `completeEquipartiteGraph` Define the complete equipartite graph in `r` parts each of *equal* size `t` such that two vertices are adjacent if and only if they are in different parts. These graphs are typically denoted by $$K_r(t)$$. --- I'm not 100% certain these definitions need their own file. I've placed them at the bottom of `CompleteMultipartite.lean` as complete equipartite graphs are just a special case of complete multipartite graphs. However, I intend to PR another definition `completeEquipartiteSubgraph`. In which case it might be appropriate to create a new file `CompleteEquipartite.lean` that contains both definitions. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-combinatorics 128/0 Mathlib/Combinatorics/SimpleGraph/Coloring.lean,Mathlib/Combinatorics/SimpleGraph/CompleteMultipartite.lean 2 1 ['github-actions'] nobody
4-20210
4 days ago
4-20956
4 days ago
4-21019
4 days
27600 ocfnash
author:ocfnash
feat: miscellaneous Lie algebra lemmas These came up in the proof that the Geck Construction yields _semisimple_ Lie algebras. I am splitting them into their own PR to simplify review. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
86/14 Mathlib/Algebra/Lie/Abelian.lean,Mathlib/Algebra/Lie/Basic.lean,Mathlib/Algebra/Lie/Semisimple/Defs.lean,Mathlib/Algebra/Lie/Subalgebra.lean 4 1 ['github-actions'] nobody
4-13045
4 days ago
4-16917
4 days ago
4-16900
4 days
27602 mitchell-horner
author:mitchell-horner
feat(Combinatorics/SimpleGraph): define `completeBipartiteSubgraph` Define the complete bipartite subgraphs of `s` and `t` parts as a "left" subset of `s` vertices and a "right" subset of `t` vertices such that every vertex in the "left" subset is adjacent to every vertex in the "right" subset. In this case `Nonempty (G.completeBipartiteSubgraph (card α) (card β))` is equivalent to `completeBipartiteGraph α β ⊑ G`, that is, finding a "left" subset of `s` vertices and a "right" subset of `t` vertices such that every vertex in the "left" subset is adjacent to every vertex in the "right" subset is equivalent to finding an injective homomorphism `completeBipartiteGraph α β` to `G`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics 88/0 Mathlib/Combinatorics/SimpleGraph/Bipartite.lean 1 1 ['github-actions'] nobody
4-12274
4 days ago
4-13909
4 days ago
4-13959
4 days
27467 themathqueen
author:themathqueen
chore(LinearAlgebra/BilinearMap): semi-linearize Semi-linearizes `llcomp` and creates a new definition `compr₂ₛₗ` for the semi-linear version of `compr₂`. Original PRs: #27353 (#27310, #24208). Co-authored-by: @ADedecker --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) maintainer-merge t-algebra
label:t-algebra$
78/30 Mathlib/Algebra/Module/Equiv/Defs.lean,Mathlib/LinearAlgebra/BilinearMap.lean 2 16 ['eric-wieser', 'github-actions', 'j-loreaux', 'themathqueen'] nobody
4-1145
4 days ago
4-1145
4 days ago
6-20557
6 days
27076 Komyyy
author:Komyyy
refactor: don't require `DecidablePred` to state `PrimrecPred` ```lean def PrimrecPred {α} [Primcodable α] (p : α → Prop) [DecidablePred p] := Primrec fun a => decide (p a) ``` Currently, `DecidablePred` is required to **state** `PrimrecPred`, so this PR changes the definition and adds convenient APIs for this new definition: ```lean def PrimrecPred {α} [Primcodable α] (p : α → Prop) := open scoped Classical in Primrec fun a => decide (p a) ``` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-computability 117/67 Mathlib/Computability/Halting.lean,Mathlib/Computability/Partrec.lean,Mathlib/Computability/Primrec.lean,Mathlib/Computability/Reduce.lean 4 8 ['Komyyy', 'digama0', 'eric-wieser', 'github-actions'] nobody
3-73946
3 days ago
19-21931
19 days ago
19-21916
19 days
22043 YaelDillies
author:YaelDillies
chore: shortcut instance for `Neg ℤˣ` This lets us avoid importing `Ring` in downstream files (most of the effect is to come). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) file-removed t-algebra
label:t-algebra$
20/47 Mathlib.lean,Mathlib/Algebra/GCDMonoid/Nat.lean,Mathlib/Algebra/Group/Int/Units.lean,Mathlib/Algebra/Order/Ring/Abs.lean,Mathlib/Algebra/Ring/Int/Units.lean,Mathlib/Algebra/Ring/NegOnePow.lean,Mathlib/Data/Fintype/Units.lean,Mathlib/Data/Int/AbsoluteValue.lean,Mathlib/Data/Int/Associated.lean,Mathlib/GroupTheory/HNNExtension.lean,Mathlib/NumberTheory/NumberField/Basic.lean,MathlibTest/Zify.lean 12 16 ['YaelDillies', 'eric-wieser', 'github-actions', 'j-loreaux', 'leanprover-community-bot-assistant', 'mathlib-bors'] nobody
3-62101
3 days ago
79-29752
2 months ago
164-2784
164 days
27301 js2357
author:js2357
feat: `MeasureTheory.Measure.sum_restrict_le` Prove that `Measure.sum (fun i ↦ μ.restrict (s i)) ≤ M • μ.restrict (⋃ i, s i)`, if at most `M` of the `s i` overlap at a single point. Also add `restrict_biUnion_le`, which is a straightforward biUnion version of the existing `restrict_iUnion_le`. Done for the Carleson project. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) carleson t-measure-probability 78/0 Mathlib/MeasureTheory/Measure/Restrict.lean 1 3 ['RemyDegenne', 'github-actions', 'js2357'] nobody
3-61214
3 days ago
3-61214
3 days ago
11-85924
11 days
27385 grunweg
author:grunweg
feat: weaken definiteness requirement for `ENormed(Add)(Comm)Monoid`s Most lemmas about these do not require the enorm to be positive definite (i.e., work fine if a nontrivial element has zero enorm), or can be rephrased easily. A handful of lemmas do require this condition. Weaken the definition of `ENormed(Add)(Comm)Monoid`s to only ask that zero have enorm zero, and add new classes `StrictENormed(Add)(Comm)Monoid` which also ask for definiteness. Most existing lemmas are kept unchanged (i.e., have slightly weaker hypotheses now); a few have their typeclasses adjusted. The motivating example behind this is `eLpNorm`, which is an enormed commutative (additive) monoid --- when we drop the definiteness requirement. This will (hopefully) allow unifying many lemma about `eLpNorm` with their more general enorm variants. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) carleson t-analysis 94/39 Mathlib/Analysis/Normed/Group/Basic.lean,Mathlib/Analysis/Normed/Group/Continuity.lean,Mathlib/Analysis/NormedSpace/PiTensorProduct/InjectiveSeminorm.lean,Mathlib/MeasureTheory/Function/LpSeminorm/Basic.lean,Mathlib/MeasureTheory/Integral/IntegrableOn.lean,Mathlib/MeasureTheory/Integral/IntervalIntegral/Basic.lean 6 5 ['github-actions', 'grunweg', 'sgouezel'] nobody
3-50220
3 days ago
8-8802
8 days ago
8-8786
8 days
27633 Ruben-VandeVelde
author:Ruben-VandeVelde
feat: MvPolynomial.coeff_mapRange --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
5/5 Mathlib/Algebra/MvPolynomial/Basic.lean,Mathlib/Algebra/MvPolynomial/Eval.lean 2 1 ['github-actions'] nobody
3-38507
3 days ago
3-38511
3 days ago
3-38560
3 days
26099 grunweg
author:grunweg
feat: add IsEmbedding.sumElim_of_separatingNhds Characterise when the Sum.elim of two inducing maps resp. embeddings is an embedding, and deduce that the ranges of the two maps lying in separated neighbourhoods suffices. This is used in my bordism theory project. Co-authored by: @plp127 --- This PR was manually re-created (and migrated to a fork at the same time) from #22137, since that seemed easiest. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-topology 103/0 Mathlib/Data/Sum/Basic.lean,Mathlib/Topology/Constructions/SumProd.lean 2 6 ['ADedecker', 'github-actions', 'grunweg'] nobody
3-34299
3 days ago
44-25473
1 month ago
44-25464
44 days
27605 ocfnash
author:ocfnash
feat: basic linear algebra lemmas about matrices These came up in the proof that the Geck Construction yields semisimple Lie algebras. I am splitting them into their own PR to simplify review. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
112/6 Mathlib/Analysis/Normed/Module/FiniteDimension.lean,Mathlib/Data/Matrix/Block.lean,Mathlib/Data/Matrix/Diagonal.lean,Mathlib/Data/Matrix/Mul.lean,Mathlib/LinearAlgebra/Basis/Basic.lean,Mathlib/LinearAlgebra/Basis/Defs.lean,Mathlib/LinearAlgebra/Eigenspace/Basic.lean,Mathlib/LinearAlgebra/Eigenspace/Matrix.lean,Mathlib/LinearAlgebra/Matrix/BilinearForm.lean,Mathlib/LinearAlgebra/Matrix/ToLin.lean,Mathlib/LinearAlgebra/Pi.lean 11 9 ['github-actions', 'j-loreaux', 'ocfnash', 'themathqueen'] nobody
3-33198
3 days ago
3-33198
3 days ago
3-51312
3 days
27008 oliver-butterley
author:oliver-butterley
feat(Dynamics): add `comp_iterate_integrable` If an observable is integrable then the observable formed by composing with iterates of a measure preserving map is also integrable. Co-authored-by: Lua Viana Reis me@lua.blog.br --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-dynamics 34/0 Mathlib.lean,Mathlib/Dynamics/MeasurePreserving/Lemmas.lean 2 1 ['github-actions'] nobody
3-31958
3 days ago
3-32022
3 days ago
21-15322
21 days
27471 FrankieNC
author:FrankieNC
feat(Topology/Baire/Lemmas): In a nonempty Baire space, any dense GDelta set is not meagre Proves that in a nonempty Baire space any dense Gδ set is not meagre --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology 7/0 Mathlib/Topology/Baire/Lemmas.lean 1 2 ['FrankieNC', 'github-actions'] nobody
3-30004
3 days ago
7-27334
7 days ago
7-27385
7 days
27635 Ruben-VandeVelde
author:Ruben-VandeVelde
chore: deprecate SubsemiringClass.coe_pow --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 2/7 Mathlib/Algebra/Ring/Subsemiring/Defs.lean,Mathlib/Analysis/Normed/Ring/Basic.lean 2 3 ['Ruben-VandeVelde', 'github-actions', 'grunweg'] nobody
3-29523
3 days ago
3-29523
3 days ago
3-32521
3 days
27320 Jlh18
author:Jlh18
doc (CategoryTheory/Bicategory/Grothendieck): rename Grothendieck to coGrothendieck Rename `CategoryTheory.Pseudofunctor.Grothendieck` to `CategoryTheory.Pseudofunctor.coGrothendieck`. Currently there are two inconsistent conventions taken in [`CategoryTheory.Grothendieck`](https://leanprover-community.github.io/mathlib4_docs/Mathlib/CategoryTheory/Grothendieck.html#CategoryTheory.Grothendieck) and [`CategoryTheory.Pseudofunctor.Grothendieck`](https://leanprover-community.github.io/mathlib4_docs/Mathlib/CategoryTheory/Bicategory/Grothendieck.html#CategoryTheory.Pseudofunctor.Grothendieck), namely the latter includes an `op` on the indexing category / base category of the Grothendieck construction. Later on, I will make more PRs to introduce the version of `CategoryTheory.Pseudofunctor.Grothendieck` that does not have an `op`. Zulip discussion: [#mathlib4 > Refactor Grothendieck from Pseudofunctor.Grothendieck](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Refactor.20Grothendieck.20from.20Pseudofunctor.2EGrothendieck/with/529165679). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-category-theory 46/38 Mathlib/CategoryTheory/Bicategory/Grothendieck.lean,Mathlib/CategoryTheory/FiberedCategory/Grothendieck.lean 2 5 ['Jlh18', 'github-actions', 'joelriou', 'kckennylau'] nobody
3-28527
3 days ago
3-28677
3 days ago
9-43719
9 days
27636 Louddy
author:Louddy
feat(Bivariate): aevalAeval and swap Add the `aeval` equivalent to `Bivariate.evalEval`. This PR also introduces `Bivariate.swap`, the R-algebra automorphism given by `X ↦ Y` and `Y ↦ X`. Co-authored-by: María Inés de Frutos Fernández <[mariaines.dff@gmail.com](mailto:mariaines.dff@gmail.com)> --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
45/0 Mathlib/Algebra/Polynomial/Bivariate.lean 1 1 ['github-actions'] nobody
3-26795
3 days ago
3-26842
3 days ago
3-26850
3 days
26842 oliver-butterley
author:oliver-butterley
feat(Mathlib/Dynamics/BirkhoffSum/Average): add lemma `birkhoffAverage_of_invariant` If a function `g` is invariant under a function `f` (i.e., `g ∘ f = g`), then the Birkhoff average of `g` over `f` for `n` iterations is equal to `g`. Requires that `0 < n`. Co-authored-by: Lua Viana Reis - [x] depends on: #26810 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor easy 10/0 Mathlib/Dynamics/BirkhoffSum/Average.lean 1 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
3-26130
3 days ago
3-26153
3 days ago
3-27040
3 days
27006 zhikaip
author:zhikaip
refactor: crossProduct notation Replace `×₃` with `⨯` (`\X` or `\crossproduct`), and manually deprecate the old syntax. See [#mathlib4 > Notation for crossProduct](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Notation.20for.20crossProduct/with/520119542) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data new-contributor t-meta 37/22 Mathlib/Geometry/Euclidean/Angle/Unoriented/CrossProduct.lean,Mathlib/LinearAlgebra/CrossProduct.lean 2 10 ['eric-wieser', 'github-actions', 'j-loreaux', 'kmill', 'madvorak'] nobody
3-25590
3 days ago
21-7214
21 days ago
21-17239
21 days
27639 staroperator
author:staroperator
feat(Algebra/Order/Sub): `Sub` instance for linearly canonically ordered monoid There is a `Sub` instance for linearly canonically ordered monoid using choice that satisfies `OrderedSub`. --- Thanks @eric-wieser for the suggestion in #27341! [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
28/0 Mathlib/Algebra/Order/Sub/Basic.lean 1 1 ['github-actions'] nobody
3-25047
3 days ago
3-25058
3 days ago
3-25104
3 days
26358 plp127
author:plp127
feat(Topology): R1 spaces are quasisober This PR continues the work from #24054. Original PR: https://github.com/leanprover-community/mathlib4/pull/24054 t-topology 24/9 Mathlib/Topology/Separation/Hausdorff.lean,Mathlib/Topology/Sober.lean 2 20 ['faenuccio', 'github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'plp127'] nobody
3-23054
3 days ago
3-27561
3 days ago
38-27752
38 days
27598 ocfnash
author:ocfnash
feat: a finite union of proper submodules is a proper subset (provided the coefficients are a sufficiently large field). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
135/1 Mathlib.lean,Mathlib/Algebra/Module/Submodule/Union.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/Data/Finset/Card.lean,Mathlib/Data/Set/Card.lean 5 1 ['github-actions'] nobody
3-22274
3 days ago
4-18663
4 days ago
4-18646
4 days
25774 Parcly-Taxel
author:Parcly-Taxel
chore: deprime `induction` in `AlgebraicTopology/CategoryTheory` Most replacements that are also in #23676 have been copied over, but some have been optimised further. tech debt 130/121 Mathlib/AlgebraicTopology/DoldKan/Decomposition.lean,Mathlib/AlgebraicTopology/DoldKan/Degeneracies.lean,Mathlib/AlgebraicTopology/DoldKan/NCompGamma.lean,Mathlib/AlgebraicTopology/DoldKan/Projections.lean,Mathlib/AlgebraicTopology/SimplexCategory/MorphismProperty.lean,Mathlib/AlgebraicTopology/SimplicialObject/Split.lean,Mathlib/AlgebraicTopology/SimplicialSet/Degenerate.lean,Mathlib/AlgebraicTopology/SimplicialSet/NerveAdjunction.lean,Mathlib/AlgebraicTopology/SimplicialSet/StdSimplex.lean,Mathlib/CategoryTheory/Abelian/GrothendieckCategory/EnoughInjectives.lean,Mathlib/CategoryTheory/Abelian/GrothendieckCategory/Subobject.lean,Mathlib/CategoryTheory/Action/Concrete.lean,Mathlib/CategoryTheory/Action/Monoidal.lean,Mathlib/CategoryTheory/ComposableArrows.lean,Mathlib/CategoryTheory/Extensive.lean,Mathlib/CategoryTheory/Filtered/Basic.lean,Mathlib/CategoryTheory/Galois/Decomposition.lean,Mathlib/CategoryTheory/Galois/EssSurj.lean,Mathlib/CategoryTheory/Limits/Shapes/Equalizers.lean,Mathlib/CategoryTheory/Limits/Shapes/SequentialProduct.lean,Mathlib/CategoryTheory/Limits/VanKampen.lean,Mathlib/CategoryTheory/Quotient.lean,Mathlib/CategoryTheory/Sites/Sheaf.lean,Mathlib/CategoryTheory/Subobject/Basic.lean,Mathlib/CategoryTheory/Subobject/FactorThru.lean,Mathlib/CategoryTheory/Subobject/Lattice.lean,Mathlib/CategoryTheory/Triangulated/TStructure/Basic.lean 27 6 ['Parcly-Taxel', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'madvorak'] nobody
3-21246
3 days ago
3-21265
3 days ago
48-13756
48 days
27333 FrankieNC
author:FrankieNC
feat: in a Baire space, every nonempty open set is of second category In a Baire space, every nonempty open set is non‑meagre (of second category). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) maintainer-merge t-topology 10/0 Mathlib/Topology/Baire/Lemmas.lean 1 13 ['FrankieNC', 'b-mehta', 'github-actions', 'grunweg'] nobody
3-19029
3 days ago
3-29501
3 days ago
10-82899
10 days
27642 themathqueen
author:themathqueen
feat(Analysis/InnerProductSpace/Projection): define symmetric projections This pr defines symmetric projections (`LinearMap.IsSymmetricProjection`) which are simply symmetric idempotents. This generalizes most of the results concerning star projection operators (since it needs completeness). In a complete space, these two definitions obviously coincide. An operator `p` is a symmetric projection if and only if it equals `(range p).starProjection`. This is a more general version of [isStarProjection_iff_eq_starProjection_range](https://leanprover-community.github.io/mathlib4_docs/Mathlib/Analysis/InnerProductSpace/Adjoint.html#isStarProjection_iff_eq_starProjection_range). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis 81/19 Mathlib/Analysis/InnerProductSpace/Adjoint.lean,Mathlib/Analysis/InnerProductSpace/Projection.lean,Mathlib/Analysis/InnerProductSpace/Symmetric.lean 3 1 ['github-actions'] nobody
3-18608
3 days ago
3-19273
3 days ago
3-19326
3 days
27638 plp127
author:plp127
feat: subsingleton `ℕ` and `ℤ` modules Provide some instances `AddCommMonoid.subsingletonNatModule` and `AddCommMonoid.subsingletonIntModule`. Also move some of the theorems about `ℕ` and `ℤ` modules from `Algebra/Module/End` to `Algebra/Module/NatInt`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
53/45 Mathlib/Algebra/Algebra/Rat.lean,Mathlib/Algebra/Module/End.lean,Mathlib/Algebra/Module/NatInt.lean,Mathlib/Algebra/Module/Submodule/RestrictScalars.lean,Mathlib/Data/ZMod/Basic.lean,Mathlib/RingTheory/OreLocalization/Ring.lean 6 3 ['github-actions', 'plp127'] nobody
3-18319
3 days ago
3-25521
3 days ago
3-25566
3 days
27634 agjftucker
author:agjftucker
fix(Analysis/Calculus/Implicit): consistently rename {`map`, `fun`, `function`} to `fun` There are several clear naming issues in the file Implicit.lean, such as ``` theorem prod_map_implicitFunction : ∀ᶠ p : F × G in 𝓝 (φ.prodFun φ.pt), φ.prodFun (φ.implicitFunction p.1 p.2) = p := ``` where `prod_map` and `prodFun` both refer to the same thing. In this PR I have done my best to resolve these as consistently as possible by renaming everything `map`, also everything `function`, to `fun`. This has the added benefit of making some long names a little shorter. In passing I rewrapped some comments and replaced `haveI` with `have` where it had been used like `haveI` in Lean 3. Moves: - ImplicitFunctionData -> ImplicitFunData - ImplicitFunctionData.implicitFunction -> ImplicitFunData.implicitFun - ImplicitFunctionData.prod_map_implicitFunction -> ImplicitFunData.prodFun_implicitFun - ImplicitFunctionData.left_map_implicitFunction -> ImplicitFunData.leftFun_implicitFun - ImplicitFunctionData.right_map_implicitFunction -> ImplicitFunData.rightFun_implicitFun - ImplicitFunctionData.implicitFunction_apply_image -> ImplicitFunData.implicitFun_apply_image - ImplicitFunctionData.implicitFunction_hasStrictFDerivAt -> ImplicitFunData.hasStrictFDerivAt_implicitFun - HasStrictFDerivAt.implicitFunctionDataOfComplemented -> HasStrictFDerivAt.implicitFunDataOfComplemented - HasStrictFDerivAt.implicitFunctionOfComplemented -> HasStrictFDerivAt.implicitFunOfComplemented - HasStrictFDerivAt.map_implicitFunctionOfComplemented_eq -> HasStrictFDerivAt.map_implicitFunOfComplemented_eq - HasStrictFDerivAt.eq_implicitFunctionOfComplemented -> HasStrictFDerivAt.eq_implicitFunOfComplemented - HasStrictFDerivAt.implicitFunctionOfComplemented_apply_image -> HasStrictFDerivAt.implicitFunOfComplemented_apply_image - HasStrictFDerivAt.to_implicitFunctionOfComplemented -> HasStrictFDerivAt.to_implicitFunOfComplemented - HasStrictFDerivAt.implicitFunction -> HasStrictFDerivAt.implicitFun - HasStrictFDerivAt.tendsto_implicitFunction -> HasStrictFDerivAt.tendsto_implicitFun - _root_.Filter.Tendsto.implicitFunction -> _root_.Filter.Tendsto.implicitFun - HasStrictFDerivAt.map_implicitFunction_eq -> HasStrictFDerivAt.map_implicitFun_eq - HasStrictFDerivAt.implicitFunction_apply_image -> HasStrictFDerivAt.implicitFun_apply_image - HasStrictFDerivAt.eq_implicitFunction -> HasStrictFDerivAt.eq_implicitFun - HasStrictFDerivAt.to_implicitFunction -> HasStrictFDerivAt.to_implicitFun --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis easy 165/121 Mathlib/Analysis/Calculus/Implicit.lean,docs/1000.yaml,docs/overview.yaml,docs/undergrad.yaml 4 1 ['github-actions'] nobody
3-13432
3 days ago
3-34878
3 days ago
3-34926
3 days
27649 hrmacbeth
author:hrmacbeth
chore: deduplicate "recursively on atoms" code This PR abstracts the "run recursively on atoms" method, implicit in `ring_nf` and `atom_nf`, for stand-alone use. The key function produced is ```lean def Mathlib.Tactic.AtomM.recurse (s : IO.Ref AtomM.State) (cfg : AtomM.Recurse.Config) (eval : Expr → AtomM Simp.Result) (cleanup : Simp.Result → MetaM Simp.Result) (tgt : Expr) : MetaM Simp.Result ``` which runs an input metaprogram `(eval : Expr → AtomM Simp.Result)` on an input expression `tgt` *recursively*: on each atom for the metaprogram `eval`, before packaging it as an atom, it finds the maximal subexpressions of that atom on which `eval` is applicable, and runs `eval` there too (and so on). Also rewrite `ring_nf` and `atom_nf` to use the abstracted method. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta 190/131 Mathlib.lean,Mathlib/Tactic/Abel.lean,Mathlib/Tactic/Ring/RingNF.lean,Mathlib/Util/AtomM/Recurse.lean,MathlibTest/ring.lean 5 1 ['github-actions'] nobody
3-327
3 days ago
3-342
3 days ago
3-2509
3 days
27655 euprunin
author:euprunin
chore(Geometry/RingedSpace): remove use of `erw` in `ofRestrict_top_c` t-algebraic-geometry 1/3 Mathlib/Geometry/RingedSpace/PresheafedSpace.lean 1 1 ['github-actions'] nobody
2-83573
2 days ago
2-83576
2 days ago
2-83622
2 days
27656 euprunin
author:euprunin
chore(Geometry/RingedSpace): remove use of `erw` in `stalkSpecializes_stalkMap` t-algebraic-geometry 1/2 Mathlib/Geometry/RingedSpace/Stalks.lean 1 1 ['github-actions'] nobody
2-83235
2 days ago
2-83248
2 days ago
2-83292
2 days
27657 euprunin
author:euprunin
chore(Geometry/RingedSpace): remove use of `erw` in `forget_preservesLimitsOfLeft` t-algebraic-geometry 5/2 Mathlib/Geometry/RingedSpace/OpenImmersion.lean 1 1 ['github-actions'] nobody
2-82890
2 days ago
2-82902
2 days ago
2-82948
2 days
27658 euprunin
author:euprunin
chore(Geometry/RingedSpace): remove use of `erw` in `app_inv_app'` t-algebraic-geometry 3/1 Mathlib/Geometry/RingedSpace/OpenImmersion.lean 1 1 ['github-actions'] nobody
2-82578
2 days ago
2-82583
2 days ago
2-82628
2 days
27659 euprunin
author:euprunin
chore(Geometry/RingedSpace): remove use of `erw` in `vPullbackConeIsLimit` t-algebraic-geometry 4/1 Mathlib/Geometry/RingedSpace/PresheafedSpace/Gluing.lean 1 1 ['github-actions'] nobody
2-82195
2 days ago
2-82200
2 days ago
2-82244
2 days
27660 euprunin
author:euprunin
chore(Geometry/RingedSpace): remove use of `erw` in `isUnit_of_isUnit_germ` t-algebraic-geometry 2/3 Mathlib/Geometry/RingedSpace/Basic.lean 1 1 ['github-actions'] nobody
2-81966
2 days ago
2-81992
2 days ago
2-82040
2 days
27665 pechersky
author:pechersky
chore(Algebra/Group/WithOne): With{One,Zero}.coe_injective --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra easy
label:t-algebra$
4/0 Mathlib/Algebra/Group/WithOne/Defs.lean 1 1 ['github-actions'] nobody
2-60360
2 days ago
2-60534
2 days ago
2-60530
2 days
26689 euprunin
author:euprunin
chore: golf Combinatorics/ using `grind` t-combinatorics 9/62 Mathlib/Combinatorics/Enumerative/Composition.lean,Mathlib/Combinatorics/Enumerative/DyckWord.lean,Mathlib/Combinatorics/Hall/Finite.lean,Mathlib/Combinatorics/SimpleGraph/Connectivity/WalkCounting.lean,Mathlib/Combinatorics/SimpleGraph/Paths.lean,Mathlib/Combinatorics/SimpleGraph/Subgraph.lean,Mathlib/Combinatorics/SimpleGraph/Trails.lean,Mathlib/Combinatorics/SimpleGraph/Triangle/Counting.lean 8 9 ['bryangingechen', 'euprunin', 'github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'leanprover-community-mathlib4-bot'] nobody
2-58095
2 days ago
24-80380
24 days ago
29-10822
29 days
26640 euprunin
author:euprunin
chore: golf Data/ using `grind` t-data 13/96 Mathlib/Data/EReal/Operations.lean,Mathlib/Data/List/Cycle.lean,Mathlib/Data/List/Indexes.lean,Mathlib/Data/List/Induction.lean,Mathlib/Data/List/Nodup.lean,Mathlib/Data/List/Permutation.lean,Mathlib/Data/List/Sigma.lean,Mathlib/Data/PEquiv.lean,Mathlib/Data/PNat/Xgcd.lean,Mathlib/Data/Prod/Lex.lean,Mathlib/Data/Seq/Parallel.lean,Mathlib/Data/Set/Lattice.lean 12 20 ['euprunin', 'github-actions', 'grunweg', 'leanprover-bot', 'leanprover-community-mathlib4-bot'] nobody
2-58017
2 days ago
7-2800
7 days ago
30-4957
30 days
26840 oliver-butterley
author:oliver-butterley
feat(Mathlib/Dynamics/BirkhoffSum/Average): add 3 BirkhoffAverage lemmas - `birkhoffAverage_add` - `birkhoffAverage_neg` - `birkhoffAverage_sub` - `birkhoffSum_add'` - `birkhoffSum_neg` - `birkhoffSum_sub` Co-authored-by: Lua Viana Reis --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-dynamics 34/1 Mathlib/Dynamics/BirkhoffSum/Average.lean,Mathlib/Dynamics/BirkhoffSum/Basic.lean 2 5 ['ADedecker', 'estradilua', 'github-actions', 'oliver-butterley'] nobody
2-51969
2 days ago
3-30568
3 days ago
25-49864
25 days
26899 robin-carlier
author:robin-carlier
feat(CategoryTheory/Functor/KanExtension): transitivity of left Kan extensions In this PR, we show that left Kan extensions are "transitive" in the following sense : if `α : F₀ ⟶ L ⋙ F₁` exhibits `F₁` as a left Kan extension of `F₀` along `L : C ⥤ D`, then given a functor `L' : D ⥤ D'` an an extension `(β : F₁ ⟶ L' ⋙ F₂)`, the "pasted extension" formed by `α` and `β` exhibits `F₂` as a left Kan extension of `F₀` along `L ⋙ L'` if and only if `β` exhibits `F₂` as a left Kan extension of `F₁` along `L'`. This refines the current theorems in mathlib that only treat the case where we pre or post-compose by an equivalence. The actual statement we prove is "fully weak" and lets us pick a functor isomorphic to `L ⋙ L'` and an extension isomorphic to the pasted one if needed. --- I will PR the dual version of everything for right Kan extensions as soon as we settle on the final form of this one. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory 144/0 Mathlib/CategoryTheory/Functor/KanExtension/Basic.lean 1 9 ['github-actions', 'joelriou', 'robin-carlier'] nobody
2-45610
2 days ago
2-45610
2 days ago
19-75703
19 days
27641 FormulaRabbit81
author:FormulaRabbit81
feat: Proof of relative compactness implies tightness of a set of measures (Easy direction of Prokhorov's theorem). PR proving the easy direction of Prokhorov's theorem. I am not sure about the naming conventions and any comments are appreciated. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import new-contributor t-measure-probability 260/1 Mathlib/Analysis/SpecificLimits/Basic.lean,Mathlib/Data/ENNReal/Operations.lean,Mathlib/MeasureTheory/Measure/ProbabilityMeasure.lean,Mathlib/MeasureTheory/Measure/Tight.lean 4 3 ['FormulaRabbit81', 'github-actions', 'themathqueen'] nobody
2-37629
2 days ago
2-57627
2 days ago
3-22467
3 days
27681 sgouezel
author:sgouezel
feat: one implication of portmanteau theorem for countably generated filters Also weaken a few assumptions in this file from metric spaces to metrizable spaces. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-measure-probability 48/8 Mathlib/MeasureTheory/Measure/Portmanteau.lean 1 1 ['github-actions'] nobody
2-31235
2 days ago
2-31243
2 days ago
2-31292
2 days
27682 FernandoChu
author:FernandoChu
Chore: Added `vecAppend_empty` lemma Added the `vecAppend_empty`. t-data new-contributor 5/0 Mathlib/Data/Fin/VecNotation.lean 1 1 ['github-actions'] nobody
2-27668
2 days ago
2-27668
2 days ago
2-27878
2 days
27549 Ruben-VandeVelde
author:Ruben-VandeVelde
feat: Submodule.smul_one_eq_span Co-authored-by: Aaron Hill Co-authored-by: Austin Letson Co-authored-by: Matej Penciak --- From FLT [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) FLT t-algebra easy
label:t-algebra$
3/0 Mathlib/Algebra/Algebra/Operations.lean 1 3 ['github-actions', 'ocfnash'] nobody
2-23812
2 days ago
5-22916
5 days ago
5-22963
5 days
27685 ocfnash
author:ocfnash
feat: add `Pi.evalLinear` (evaluation as a linear map) --- I'm amazed this seems not to exist already but I can't find it after looking carefully. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-algebra easy
label:t-algebra$
24/1 Mathlib/Algebra/Module/Pi.lean,Mathlib/Order/Filter/Germ/Basic.lean 2 1 ['github-actions'] nobody
2-23172
2 days ago
2-24507
2 days ago
2-25287
2 days
27556 kebekus
author:kebekus
feat: analyticity of harmonic functions, Part I If `f : ℂ → ℝ` is harmonic at `x`, show that `∂f/∂1 - I • ∂f/∂I` is complex-analytic at `x`. As soon as PR #9598 (feat(Analysis/Complex): HasPrimitives on disc) is merged, I will extend this result to show that `f` itself is locally the real part of a holomorphic function, and hence real-analytic. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis 66/0 Mathlib.lean,Mathlib/Analysis/InnerProductSpace/Harmonic/Analytic.lean 2 3 ['github-actions', 'kebekus', 'sgouezel'] nobody
2-11604
2 days ago
5-14124
5 days ago
5-14168
5 days
24730 YaelDillies
author:YaelDillies
feat(RingTheory): group-like elements Define group-like elements in a bialgebra, ie elements such that `η a = 1` and `Δ a = a ⊗ₜ a`. We prove that group-like elements of a coalgebra over a domain are linearly independent, group-like elements of a bialgebra form a monoid, group-like elements of a Hopf algebra form a group. From Toric Co-authored-by: Michał Mrugała --- - [x] depends on: #24747 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) toric t-algebra
label:t-algebra$
309/0 Mathlib.lean,Mathlib/RingTheory/Bialgebra/GroupLike.lean,Mathlib/RingTheory/Coalgebra/GroupLike.lean,Mathlib/RingTheory/HopfAlgebra/GroupLike.lean 4 33 ['Julian-Kuelshammer', 'Parcly-Taxel', 'YaelDillies', 'erdOne', 'eric-wieser', 'github-actions', 'leanprover-bot', 'mathlib4-dependent-issues-bot', 'smorel394'] eric-wieser
assignee:eric-wieser
2-7095
2 days ago
82-85041
2 months ago
83-194
83 days
24998 YaelDillies
author:YaelDillies
chore(Algebra/Notation): separate very basic lemmas about `Set.indicator` and `Pi.single` The very basic lemmas go under `Algebra.Notation` and do not import `Monoid`. This is useful to disentangle `Finsupp` results downstream. --- - [x] depends on: #25040 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) file-removed 719/640 Mathlib.lean,Mathlib/Algebra/BigOperators/Finprod.lean,Mathlib/Algebra/BigOperators/Group/Finset/Lemmas.lean,Mathlib/Algebra/BigOperators/GroupWithZero/Finset.lean,Mathlib/Algebra/BigOperators/Pi.lean,Mathlib/Algebra/Divisibility/Prod.lean,Mathlib/Algebra/Group/End.lean,Mathlib/Algebra/Group/Equiv/TypeTags.lean,Mathlib/Algebra/Group/Fin/Tuple.lean,Mathlib/Algebra/Group/Finsupp.lean,Mathlib/Algebra/Group/Hom/Defs.lean,Mathlib/Algebra/Group/Indicator.lean,Mathlib/Algebra/Group/Nat/Hom.lean,Mathlib/Algebra/Group/NatPowAssoc.lean,Mathlib/Algebra/Group/Pi/Basic.lean,Mathlib/Algebra/Group/Pointwise/Set/Scalar.lean,Mathlib/Algebra/Group/Prod.lean,Mathlib/Algebra/Group/Support.lean,Mathlib/Algebra/Group/TypeTags/Basic.lean,Mathlib/Algebra/GroupWithZero/Action/Defs.lean,Mathlib/Algebra/GroupWithZero/Indicator.lean,Mathlib/Algebra/Homology/Additive.lean,Mathlib/Algebra/Module/Basic.lean,Mathlib/Algebra/Notation/FiniteSupport.lean,Mathlib/Algebra/Notation/Indicator.lean,Mathlib/Algebra/Notation/Pi/Basic.lean,Mathlib/Algebra/Notation/Pi/Defs.lean,Mathlib/Algebra/Notation/Support.lean,Mathlib/Algebra/Order/Field/Pi.lean,Mathlib/Algebra/Order/Group/Unbundled/Abs.lean,Mathlib/Algebra/Order/GroupWithZero/Unbundled/Basic.lean,Mathlib/Algebra/Order/Sub/Prod.lean,Mathlib/Algebra/Order/Sum.lean,Mathlib/Algebra/Ring/CharZero.lean,Mathlib/Algebra/Ring/Hom/Defs.lean,Mathlib/CategoryTheory/Limits/Shapes/ZeroMorphisms.lean,Mathlib/Combinatorics/Additive/Dissociation.lean,Mathlib/Combinatorics/SimpleGraph/Bipartite.lean,Mathlib/Data/Finsupp/Basic.lean,Mathlib/Data/Finsupp/Defs.lean,Mathlib/Data/Finsupp/Single.lean,Mathlib/Data/Int/CharZero.lean,Mathlib/Data/Set/Pointwise/Support.lean,Mathlib/GroupTheory/FreeGroup/Basic.lean,Mathlib/MeasureTheory/MeasurableSpace/Basic.lean,Mathlib/Order/Filter/Basic.lean,Mathlib/Order/Filter/EventuallyConst.lean,Mathlib/Order/Interval/Set/Pi.lean,Mathlib/RingTheory/HahnSeries/Addition.lean,Mathlib/RingTheory/HahnSeries/Basic.lean,Mathlib/Topology/Algebra/Indicator.lean,Mathlib/Topology/IndicatorConstPointwise.lean,Mathlib/Topology/LocallyConstant/Basic.lean,Mathlib/Topology/LocallyFinsupp.lean,Mathlib/Topology/Separation/Basic.lean,Mathlib/Topology/Separation/DisjointCover.lean 56 13 ['YaelDillies', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] ericrbg
assignee:ericrbg
2-7094
2 days ago
26-46827
26 days ago
66-83576
66 days
25123 eric-wieser
author:eric-wieser
feat: add rfl lemmas for monoidal categories Making these `simp` opens a can of worms best left to #24823 `simps` would generate bad names here. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
111/0 Mathlib/Algebra/Category/AlgCat/Monoidal.lean,Mathlib/Algebra/Category/ModuleCat/Monoidal/Basic.lean,Mathlib/LinearAlgebra/QuadraticForm/QuadraticModuleCat/Monoidal.lean 3 1 ['github-actions'] dagurtomas
assignee:dagurtomas
2-7093
2 days ago
70-73656
2 months ago
70-73706
70 days
25401 digama0
author:digama0
feat(Util): SuppressSorry option See also leanprover/lean4#8611 and [#lean4 > Silent sorry @ 💬](https://leanprover.zulipchat.com/#narrow/channel/270676-lean4/topic/Silent.20sorry/near/503537964). This is a stop-gap solution while leanprover/lean4#8611 is underway, but it works about as well as any other built in option. Hooking declaration elaborators turns out to be a very powerful technique. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta 342/0 Mathlib.lean,Mathlib/Util/CommandElabHook.lean,Mathlib/Util/SuppressSorry.lean,MathlibTest/suppressSorry.lean 4 13 ['digama0', 'eric-wieser', 'github-actions'] alexjbest
assignee:alexjbest
2-7092
2 days ago
58-11648
1 month ago
59-21994
59 days
25864 plp127
author:plp127
feat(Nat/Digits): use fuel in `Nat.digits` Add a `fuel` parameter to `Nat.digitsAux` to make it structurally recursive. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data 47/14 Mathlib/Data/Nat/Digits/Defs.lean 1 2 ['github-actions', 'leanprover-community-bot-assistant'] ericrbg
assignee:ericrbg
2-7089
2 days ago
12-84165
12 days ago
33-44323
33 days
25875 robin-carlier
author:robin-carlier
feat(CategoryTheory/Monoidal/Action): actions as monoidal functors to endofunctors Given a monoidal category `C` and a category `D`, we show that left actions of `C` on `D` correspond to monoidal functors `C ⥤ (D ⥤ D)ᴹᵒᵖ` by showing that the composition of `curriedAction C D` with `mopFunctor` is monoidal, and in the other direction by defining an action of `C` on `D` out of the data of such a monoidal functor. Similarly, we show that monoidal functors `C ⥤ (D ⥤ D)` correspond to right actions of `C` on `D`. We use this to define the "evaluation" right action of `(C ⥤ C)` (with the composition monoidal structure) on `C` as the action corresponding to the identity functor `(C ⥤ C) ⥤ (C ⥤ C)`. --- - [x] depends on: #25840 - [x] depends on: #25766 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory 222/3 Mathlib.lean,Mathlib/CategoryTheory/Monoidal/Action/Basic.lean,Mathlib/CategoryTheory/Monoidal/Action/End.lean,Mathlib/CategoryTheory/Monoidal/Opposite.lean 4 4 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] joelriou
assignee:joelriou
2-7088
2 days ago
27-26788
27 days ago
39-77671
39 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/) t-algebraic-geometry 44/0 Mathlib/AlgebraicGeometry/EllipticCurve/Affine/Point.lean 1 10 ['MichaelStollBayreuth', 'Multramate', 'acmepjz', 'github-actions', 'kckennylau'] dagurtomas
assignee:dagurtomas
2-7087
2 days ago
44-34270
1 month ago
44-34314
44 days
26428 Ruben-VandeVelde
author:Ruben-VandeVelde
feat: norm_num support for Int.fract --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data 44/0 Mathlib/Data/Rat/Floor.lean,MathlibTest/norm_num_ext.lean 2 5 ['Rob23oba', 'github-actions'] ericrbg
assignee:ericrbg
2-7085
2 days ago
36-766
1 month ago
36-45524
36 days
26617 vihdzp
author:vihdzp
feat(Data/Sum/Order): `toLex` as a `RelIso` As [requested](https://github.com/leanprover-community/mathlib4/pull/20409#discussion_r1903319844) by @eric-wieser in #20409. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data t-order 30/0 Mathlib/Data/Sum/Order.lean 1 4 ['eric-wieser', 'github-actions', 'kckennylau', 'vihdzp'] ericrbg
assignee:ericrbg
2-7084
2 days ago
30-63808
30 days ago
30-64070
30 days
26945 gasparattila
author:gasparattila
feat(LinearAlgebra/AffineSpace/AffineSubspace): basic properties of `sInf` and `iInf` These properties are analogous to the existing ones for the binary infimum. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra
label:t-algebra$
48/1 Mathlib/LinearAlgebra/AffineSpace/AffineSubspace/Defs.lean 1 4 ['Ruben-VandeVelde', 'gasparattila', 'github-actions'] eric-wieser
assignee:eric-wieser
2-7081
2 days ago
23-11482
23 days ago
23-11528
23 days
26986 WangYiran01
author:WangYiran01
feat(Partition): add bijection for partitions with max part ≤ r ## Summary This PR adds a new theorem `partition_max_equals_bound` to `Mathlib.Combinatorics.Enumerative.Partition`. It constructs a bijection between: - The set of partitions of `n` in which `r ∈ π.parts` and all parts are `≤ r`, and - The set of partitions of `n - r` whose largest part is at most `r`. This provides a constructive proof via removing/adding `r` from/to the partition multiset, in line with classical enumerative combinatorics. ## Implementation notes - The proof uses `Multiset.erase` and `Multiset.cons` with basic properties of `sum`, `sup`, and `Partition` structures. - The bijection is implemented explicitly via `f` and `g`, and proven mutually inverse via `Subtype.ext`. ## Linting - [x] Passes `lake build` - [x] Linter clean (no commandStart or longLine issues) ## Author Contributed by Yiran Wang. new-contributor t-combinatorics 85/0 Mathlib/Combinatorics/Enumerative/Partition.lean 1 2 ['WangYiran01', 'github-actions'] b-mehta
assignee:b-mehta
2-7080
2 days ago
21-44283
21 days ago
21-44327
21 days
27664 pechersky
author:pechersky
feat(Topology,Analysis): discrete topology metric space and normed groups Explicit construction of the discrete topology metric space and normed groups where `dist x y = 1` for all `x != y` Provide PseudoMetricSpace, MetricSpace, Seminormed(Add)Group, and Normed(Add)Group constructions --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology 137/0 Mathlib/Analysis/Normed/Group/Basic.lean,Mathlib/Topology/MetricSpace/Basic.lean,Mathlib/Topology/MetricSpace/Pseudo/Constructions.lean 3 1 ['github-actions'] nobody
2-7031
2 days ago
2-64332
2 days ago
2-64325
2 days
27697 BoltonBailey
author:BoltonBailey
chore(Data/Fintype): use `univ` instead of `Fintype.elems` A short PR to keep the API consistent with its surroundings. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data 2/2 Mathlib/Data/Fintype/Defs.lean 1 1 ['github-actions', 'vihdzp'] nobody
2-3261
2 days ago
2-7140
2 days ago
2-7185
2 days
27238 alreadydone
author:alreadydone
feat(Algebra): IsDomain R[X] ↔ IsDomain R ∧ IsCancelAdd R --- - [x] depends on: #27241 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-algebra
label:t-algebra$
138/4 Counterexamples.lean,Counterexamples/PolynomialIsDomain.lean,Mathlib/Algebra/Group/Defs.lean,Mathlib/Algebra/Group/Opposite.lean,Mathlib/Algebra/GroupWithZero/Defs.lean,Mathlib/Algebra/GroupWithZero/TransferInstance.lean,Mathlib/Algebra/Opposites.lean,Mathlib/Algebra/Polynomial/Basic.lean,Mathlib/RingTheory/Polynomial/Opposites.lean 9 6 ['alreadydone', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
2-1793
2 days ago
2-2161
2 days ago
2-59174
2 days
25491 tannerduve
author:tannerduve
feat(Control/Monad/Free): define free monad, prove it lawful, and implement standard effects This PR introduces the `Free` monad. This implementation uses the "freer monad" approach as the traditional free monad (eg from [Haskell](https://hackage.haskell.org/package/free-5.2/docs/Control-Monad-Free.html)) is not safely definable in Lean due to termination checking (it's not strictly positive). The main contributions are: * Definition of the `Free` monad as an inductive type which generates a monad given any type constructor `F : Type -> Type`. * Functor and Monad instances for `Free F`, along with proofs of the `LawfulFunctor` and `LawfulMonad` laws. * Canonical instances of `Free` with standard effect signatures: * `FreeState s` for stateful computations, defined via a `StateF s` functor with `get` and `put` operations. * `FreeWriter w` for logging computations, defined via a `WriterF w` functor with a `tell` operation. * `FreeCont r` for continuation-passing computations, using the CPS functor `(α → r) → r`. In this construction, computations are represented as **trees of effects**. Each node (`liftBind`) represents a request to perform an effect, accompanied by a continuation specifying how the computation proceeds after the effect. The leaves (`pure`) represent completed computations with final results. A key insight is that `FreeM F` satisfies the **universal property of free monads**: for any monad `M` and effect handler `f : F → M`, there exists a unique way to interpret `FreeM F` computations in `M` that respects the effect semantics given by `f`. This unique interpreter is `liftM f`, which acts as the canonical **fold** for free monads. To execute or interpret these computations, we provide two approaches: 1. **Hand-written interpreters** (`FreeState.run`, `FreeWriter.run`, `FreeCont.run`) that directly pattern-match on the tree structure 2. **Canonical interpreters** (`FreeState.toStateM`, `FreeWriter.toWriteT`, `FreeCont.toContT`) derived from the universal property via `liftM` And then prove that these approaches are equivalent --- This PR adds new files and definitions; no breaking changes. **Tags:** free monad, freer monad, effect systems, state monad, writer monad, continuation monad, operational semantics, verified interpreters t-data maintainer-merge 696/0 Mathlib.lean,Mathlib/Control/Monad/Free.lean,Mathlib/Control/Monad/Free/Effects.lean,MathlibTest/freemonad.lean,docs/references.bib 5 146 ['YaelDillies', 'copilot-pull-request-reviewer', 'eric-wieser', 'github-actions', 'plp127', 'quangvdao', 'tannerduve'] nobody
1-85328
1 day ago
45-23714
1 month ago
55-42795
55 days
27015 vihdzp
author:vihdzp
feat: `aleph` and `beth` are normal functions By using `Order.IsNormal`, we can state (and use!) these results directly, instead of having to go through `ord`. --- - [x] depends on: #26900 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 58/40 Mathlib/Order/ConditionallyCompleteLattice/Indexed.lean,Mathlib/Order/IsNormal.lean,Mathlib/SetTheory/Cardinal/Aleph.lean 3 4 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
1-84946
1 day ago
1-84970
1 day ago
2-1341
2 days
26295 DavidJWebb
author:DavidJWebb
feat: filtering lists and bounded quantifiers are primitive recursive A few useful lemmas not explicitly in Primrec.lean : - Filtering for elements from a list that meet a primrec criterion is primrec - Checking whether a list has some element meeting a primrec criterion is primrec - Checking whether every element of a list meets a primrec criterion is primrec - Primitive recursive functions are closed under bounded existential and universal quantifiers --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-computability new-contributor 174/0 Mathlib.lean,Mathlib/Computability/PrimrecFilter.lean 2 65 ['DavidJWebb', 'github-actions', 'grunweg'] nobody
1-84072
1 day ago
1-84268
1 day ago
30-11783
30 days
26646 eric-wieser
author:eric-wieser
feat(TensorProduct): add a Repr Now that tensor products are computable again, this makes them `#eval`able. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-meta
label:t-algebra$
8/0 Mathlib/LinearAlgebra/TensorProduct/Basic.lean 1 7 ['JovanGerb', 'eric-wieser', 'github-actions'] kim-em
assignee:kim-em
1-76832
1 day ago
29-72324
29 days ago
29-72375
29 days
27703 vihdzp
author:vihdzp
feat: `le_of_forall_ne` This form of `le_of_forall_lt` is a bit nicer when working with nimbers; they're minimum excludents, so to prove `a ≤ b` you have to prove `b` can't be equal to any smaller `a`! --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order easy 7/0 Mathlib/Order/Basic.lean 1 1 ['github-actions'] nobody
1-76452
1 day ago
1-85686
1 day ago
1-85687
1 day
27705 yonggyuchoimath
author:yonggyuchoimath
feat(RingTheory.Ideal.Height): add trivial cases feat: add trivial cases of Ideal.Height --- This PR updates `RingTheory.Ideal.Height`, which adds two lemmas `Ideal.height_of_subsingleton` and `Ideal.height_bot_eq_zero`. These compute the height of (any) ideal in a zero commutative ring, and the height of the zero ideal in a nonzero commutative ring. new-contributor t-algebra
label:t-algebra$
9/0 Mathlib/RingTheory/Ideal/Height.lean 1 5 ['erdOne', 'github-actions', 'yonggyuchoimath'] nobody
1-71642
1 day ago
1-83096
1 day ago
1-83140
1 day
25889 plp127
author:plp127
fix(Tactic/Widget/Conv): fix various issues Fixes various issues with the `conv?` widget. Closes #25162. ([Zulip thread](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/bug.20in.20.60conv.3F.60)) Specifically, fixes issues with `conv?` where - when converting a `SubExpr.Pos` to conv directions, it always uses the goal expression as reference, even when working on a hypothesis, this often leads to bad results and makes it unusable on hypotheses - it refuses to go all the way in to a function (for example in `Nat.succ 0`, you can't access `Nat.succ`) - it refuses to enter binders where the name of the bound variable contains the character `0` (try it on `∀ (x0 : Nat), x0 = x0`) - it panics if it can't find a binder name instead of just coming up with one itself, this also means usually you can't enter either side of a non-dependent arrow since those usually don't have binder names (try it on `False → False`) - you can't enter the type of a binder, you end up going into the body instead (try it on `fun (x : False) => (x.elim : False → Nat) x.elim`) - you can't partially enter a function, you end up going to the top argument after instead (for example, in the expression `id (id id) 0`, when you click on `id (id id)`, you end up going to `id id`) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta 419/84 Mathlib/Tactic/Widget/Conv.lean,MathlibTest/conv?.lean 2 4 ['bryangingechen', 'github-actions', 'plp127'] bryangingechen
assignee:bryangingechen
1-67178
1 day ago
47-67944
1 month ago
47-67989
47 days
27712 kim-em
author:kim-em
chore: remove old irrelevant attributes in Logic/Basic This PR removes some attributes from Logic/Basic that appear to have no effect on Mathlib. t-logic 0/2 Mathlib/Logic/Basic.lean 1 4 ['github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot'] nobody
1-65587
1 day ago
1-65587
1 day ago
1-70485
1 day
27162 themathqueen
author:themathqueen
feat(Analysis/InnerProductSpace/Positive): `U.starProjection ≤ V.starProjection` iff `U ≤ V` For star projections `p` and `q`, `p ≤ q` iff `p ∘ q = p`, so then a corollary is: `U.starProjection ≤ V.starProjection` iff `U ≤ V`. --- - [x] depends on: #25910 - [x] depends on: #27619 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 37/0 Mathlib/Analysis/InnerProductSpace/Positive.lean 1 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
1-54331
1 day ago
1-56749
1 day ago
1-57541
1 day
27534 PierreQuinton
author:PierreQuinton
Add `LawfulPreorder` Adds lawful infima and suprema type classes. A preorder with lawful suprema: whenever a set has a least upper bound, `sSup` returns a least upper bound for that set. A preorder with lawful infima: whenever a set has a greatest lower bound, `sInf` returns a greastest lower bound for that set. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order 121/8 Mathlib.lean,Mathlib/Order/CompleteLattice/Defs.lean,Mathlib/Order/LawfulSupInf.lean 3 11 ['PierreQuinton', 'github-actions', 'vihdzp'] nobody
1-51027
1 day ago
5-21383
5 days ago
5-21417
5 days
27720 peabrainiac
author:peabrainiac
feat(CategoryTheory/Adjunction): lemmas on adjoint quadruples Lemmas about adjoint quadruples `L ⊣ F ⊣ G ⊣ R` where some of the functors are fully faithful: * If `F` and `R` are fully faithful, the components of the induced natural transformation `G ⟶ L` are epic iff the components of the natural transformation `F ⟶ R` are monic. * If `L` and `G` are fully faithful, the components of the induced natural transformation `L ⟶ G` are epic iff the components of the natural transformation `R ⟶ F` are monic. A variant of the first case appears as proposition 2.7 on the nlab [here](https://ncatlab.org/nlab/show/cohesive+topos); the second case is dual. From [lean-orbifolds](https://github.com/peabrainiac/lean-orbifolds/blob/d599ff5f39aa831e8fa79b2f2fa7178b36bcbafd/Orbifolds/ForMathlib/Quadruple.lean). --- Continued / revived from #24667. t-category-theory 178/0 Mathlib.lean,Mathlib/CategoryTheory/Adjunction/Quadruple.lean,Mathlib/CategoryTheory/Adjunction/Triple.lean,Mathlib/CategoryTheory/Category/Basic.lean,Mathlib/CategoryTheory/EpiMono.lean 5 2 ['github-actions', 'peabrainiac'] nobody
1-50781
1 day ago
1-52198
1 day ago
1-52904
1 day
27383 euprunin
author:euprunin
chore: replace `omega` with `grind` in `Algebra/` theorems/lemmas where applicable Motivation: `grind` subsumes `omega`, which is expected to be deprecated. t-algebra
label:t-algebra$
225/225 Mathlib/Algebra/AddConstMap/Basic.lean,Mathlib/Algebra/BigOperators/Fin.lean,Mathlib/Algebra/CharP/Defs.lean,Mathlib/Algebra/ContinuedFractions/Computation/Approximations.lean,Mathlib/Algebra/ContinuedFractions/Computation/TerminatesIffRat.lean,Mathlib/Algebra/CubicDiscriminant.lean,Mathlib/Algebra/GCDMonoid/Nat.lean,Mathlib/Algebra/GeomSum.lean,Mathlib/Algebra/Group/Defs.lean,Mathlib/Algebra/Group/Int/Even.lean,Mathlib/Algebra/Group/Nat/Range.lean,Mathlib/Algebra/GroupWithZero/Basic.lean,Mathlib/Algebra/GroupWithZero/Units/Basic.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/Basic.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/EnoughInjectives.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/EnoughProjectives.lean,Mathlib/Algebra/Homology/DerivedCategory/Fractions.lean,Mathlib/Algebra/Homology/Embedding/Basic.lean,Mathlib/Algebra/Homology/Embedding/Boundary.lean,Mathlib/Algebra/Homology/Embedding/CochainComplex.lean,Mathlib/Algebra/Homology/Embedding/Connect.lean,Mathlib/Algebra/Homology/ExactSequence.lean,Mathlib/Algebra/Homology/HomotopyCategory/HomComplex.lean,Mathlib/Algebra/Homology/HomotopyCategory/HomComplexShift.lean,Mathlib/Algebra/Homology/HomotopyCategory/Pretriangulated.lean,Mathlib/Algebra/Homology/HomotopyCategory/ShiftSequence.lean,Mathlib/Algebra/Homology/HomotopyCategory/ShortExact.lean,Mathlib/Algebra/Homology/TotalComplexShift.lean,Mathlib/Algebra/Lie/LieTheorem.lean,Mathlib/Algebra/Lie/Nilpotent.lean,Mathlib/Algebra/Lie/Sl2.lean,Mathlib/Algebra/Lie/Weights/Chain.lean,Mathlib/Algebra/Lie/Weights/Killing.lean,Mathlib/Algebra/Lie/Weights/RootSystem.lean,Mathlib/Algebra/Module/LinearMap/End.lean,Mathlib/Algebra/MvPolynomial/Degrees.lean,Mathlib/Algebra/Order/Antidiag/Nat.lean,Mathlib/Algebra/Order/Floor/Ring.lean,Mathlib/Algebra/Order/Group/Basic.lean,Mathlib/Algebra/Order/Group/Int/Sum.lean,Mathlib/Algebra/Order/Group/Unbundled/Int.lean,Mathlib/Algebra/Order/GroupWithZero/Unbundled/Basic.lean,Mathlib/Algebra/Order/Monoid/Unbundled/Pow.lean,Mathlib/Algebra/Order/Ring/Int.lean,Mathlib/Algebra/Order/Ring/Unbundled/Rat.lean,Mathlib/Algebra/Polynomial/AlgebraMap.lean,Mathlib/Algebra/Polynomial/Degree/IsMonicOfDegree.lean,Mathlib/Algebra/Polynomial/Derivative.lean,Mathlib/Algebra/Polynomial/FieldDivision.lean,Mathlib/Algebra/Polynomial/Laurent.lean,Mathlib/Algebra/Polynomial/Module/Basic.lean,Mathlib/Algebra/Polynomial/OfFn.lean,Mathlib/Algebra/Polynomial/Sequence.lean,Mathlib/Algebra/Polynomial/UnitTrinomial.lean,Mathlib/Algebra/Ring/Divisibility/Lemmas.lean,Mathlib/Algebra/Squarefree/Basic.lean,Mathlib/Algebra/Vertex/VertexOperator.lean 57 18 ['euprunin', 'github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'leanprover-community-mathlib4-bot'] nobody
1-47152
1 day ago
1-47170
1 day ago
8-80943
8 days
27339 pechersky
author:pechersky
chore(RingTheory/Laurent): use WithZero.exp to golf statements and proofs about valuation on K((X)) Done as part of refactor of Valued in #27314. This PR does not change any definitions. Instead, uses `WithZero.exp` instead of coercion + Multiplicative.ofAdd. And some helper simp lemmas about valuations of RatFunc vis a vis LaurentSeries. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) tech debt t-algebra t-number-theory
label:t-algebra$
78/77 Mathlib/FieldTheory/RatFunc/AsPolynomial.lean,Mathlib/RingTheory/LaurentSeries.lean,Mathlib/Topology/Algebra/Valued/WithVal.lean 3 1 ['github-actions'] Vierkantor
assignee:Vierkantor
1-45408
1 day ago
10-24187
10 days ago
10-68182
10 days
27738 ChrisHughes24
author:ChrisHughes24
feat(Rat): Decidable instance for IsSquare --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data 3/0 Mathlib/Data/Rat/Lemmas.lean 1 1 ['github-actions'] nobody
1-43876
1 day ago
1-43880
1 day ago
1-43927
1 day
27735 kebekus
author:kebekus
feat: mean value property of complex differentiable functions on the complex plane As an immediate application of the Cauchy integral formula, establish the mean value property of complex-differentiable functions on the complex plane. Fix a typo in the docstrings of `Mathlib/Analysis/Complex/CauchyIntegral.lean` and remove one unnecessary type cast. This material is used in [Project VD](https://github.com/kebekus/ProjectVD), which aims to formalize Value Distribution Theory for meromorphic functions on the complex plane. TODO: As soon as PR https://github.com/leanprover-community/mathlib4/pull/9598 (feat(Analysis/Complex): HasPrimitives on disc) is merged, extend this to harmonic functions. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis 99/5 Mathlib.lean,Mathlib/Analysis/Complex/CauchyIntegral.lean,Mathlib/Analysis/Complex/MeanValue.lean,Mathlib/MeasureTheory/Integral/CircleAverage.lean 4 1 ['github-actions'] nobody
1-43793
1 day ago
1-43793
1 day ago
1-46641
1 day
27739 ChrisHughes24
author:ChrisHughes24
feat(Int): Decidable instance for IsCoprime --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
3/0 Mathlib/RingTheory/Coprime/Lemmas.lean 1 1 ['github-actions'] nobody
1-43566
1 day ago
1-43576
1 day ago
1-43621
1 day
24794 chrisflav
author:chrisflav
feat(RingTheory/Presentation): core of a presentation If `P` is a presentation of `S` as an `R`-algebra and `R₀` a subring of `R` containing the coefficients of the relations of `P`, then there exists an `R₀`-algebra `S₀` such that `S` is isomorphic to the base change of `S₀` to `R`. This is a tool to remove Noetherian hypothesis in certain situations. --- - [x] depends on: #24788 - [x] depends on: #24786 - [x] depends on: #24785 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
252/2 Mathlib.lean,Mathlib/Algebra/Algebra/Subalgebra/Basic.lean,Mathlib/Algebra/Algebra/Subalgebra/Tower.lean,Mathlib/Algebra/Algebra/Tower.lean,Mathlib/RingTheory/AlgebraicIndependent/Transcendental.lean,Mathlib/RingTheory/Extension/Presentation/Core.lean,Mathlib/RingTheory/FiniteType.lean,Mathlib/RingTheory/TensorProduct/MvPolynomial.lean 8 10 ['erdOne', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] Vierkantor
assignee:Vierkantor
1-39052
1 day ago
53-47777
1 month ago
53-48715
53 days
25179 YaelDillies
author:YaelDillies
feat: `#print sorries`, a command to find usage of `sorry` `#print sorries` returns all sorries in the current file. `#print sorries id1 ... idn` returns all sorries in declarations `id1`, ..., `idn`. Such a command is a recurrent need of the community, see eg [here](https://leanprover.zulipchat.com/#narrow/channel/217875-Is-there-code-for-X.3F/topic/Hunting.20down.20axioms/with/495448595) most recently. From Toric Co-authored-by: Henrik Böving Co-authored-by: Kyle Miller --- An alternative implementation was provided in [#Is there code for X? > ✔ Finding usages of `sorry` in external code @ 💬](https://leanprover.zulipchat.com/#narrow/channel/217875-Is-there-code-for-X.3F/topic/.E2.9C.94.20Finding.20usages.20of.20.60sorry.60.20in.20external.20code/near/430509619) by @kmill. I prefer the current one because it only prints something for uses of `sorry` and not the other three standard axioms. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) toric t-meta 103/0 Mathlib.lean,Mathlib/Util/PrintSorries.lean 2 11 ['YaelDillies', 'eric-wieser', 'github-actions', 'kmill'] dwrensha
assignee:dwrensha
1-39051
1 day ago
68-47471
2 months ago
68-47521
68 days
25267 YaelDillies
author:YaelDillies
feat: `counit (antipode a) = counit a` and unsimp `sum_antipode_mul_eq_algebraMap_counit`/`sum_mul_antipode_eq_algebraMap_counit` since they are annoying lemmas to fight against. From Toric Co-authored-by: Patrick Massot --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) toric t-algebra
label:t-algebra$
51/18 Mathlib/RingTheory/Coalgebra/Basic.lean,Mathlib/RingTheory/HopfAlgebra/Basic.lean,Mathlib/RingTheory/HopfAlgebra/MonoidAlgebra.lean 3 10 ['YaelDillies', 'erdOne', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant'] chrisflav
assignee:chrisflav
1-39050
1 day ago
27-54414
27 days ago
65-7586
65 days
26155 xroblot
author:xroblot
feat(DedekindDomain/Different): add the transitivity formula This PR proves the transitivity formula for the different ideal. It introduces ~~two~~ one increase~~s~~ in imports: - `RingTheory.FractionalIdeal.Extended`: this is a short leaf file and I think the import makes sense there - ~~`RingTheory.Localization.Defs.lean `: the file `Algebra.Algebra.Basic` is added since it is necessary to have the definition of `noZeroSMulDivisors` to get that some algebra map is injective. The import could be removed by stating the hypothesis as `Function.Injective (algebraMap * *)` but it is not the usual spelling (and cannot be synthesized by Lean). In the end, it appears that the increased import only affects three files so maybe it's fine.~~ The PR also adds two new instances: - `FiniteDimensional (FractionRing A) (FractionRing B)` deduced from `Module.Finite A B` when `B` is a Dedekind domain. - `IsScalarTower (FractionRing A) (FractionRing B) (FractionRing C)` deduced from `IsScalarTower A B C` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-algebra
label:t-algebra$
207/4 Mathlib/RingTheory/DedekindDomain/Different.lean,Mathlib/RingTheory/DedekindDomain/IntegralClosure.lean,Mathlib/RingTheory/FractionalIdeal/Extended.lean,Mathlib/RingTheory/Localization/Basic.lean,Mathlib/RingTheory/Localization/FractionRing.lean 5 13 ['erdOne', 'github-actions', 'xroblot'] Vierkantor
assignee:Vierkantor
1-39048
1 day ago
35-31680
1 month ago
40-28687
40 days
26259 Raph-DG
author:Raph-DG
feat(Topology): Connecting different notions of locally finite In this PR we connect the notions of local finiteness of an indexed family of sets (as in LocallyFinite) and of a set of sets (as in Function.locallyFinsuppWithin) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology 32/0 Mathlib/Topology/LocallyFinsupp.lean 1 3 ['Raph-DG', 'github-actions', 'kckennylau'] jcommelin
assignee:jcommelin
1-39047
1 day ago
41-10402
1 month ago
41-10443
41 days
26453 jburroni
author:jburroni
feat(Data/PNat/Basic): add order-related instances to PNat Add `SuccAddOrder ℕ+` and `NoMaxOrder ℕ+` instances. This allows, for example, the use of lemmas related to `Intervals` built with ℕ+. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-data new-contributor 18/0 Mathlib/Data/PNat/Basic.lean 1 3 ['eric-wieser', 'github-actions', 'jburroni'] ericrbg
assignee:ericrbg
1-39046
1 day ago
36-10867
1 month ago
36-10911
36 days
26645 erdOne
author:erdOne
feat(RingTheory/PowerSeries): Construction of `Q` such that `P(Q(X)) = X` Co-authored-by: Junnosuke Koizumi Co-authored-by: Hyeon, Seung-Hyeon Co-authored-by: Yuichiro Taguchi This contribution was created as part of the ZMC conference 2025 "Anabelian Geometry and its Computer Formalization". --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
133/0 Mathlib/RingTheory/PowerSeries/Substitution.lean 1 9 ['chrisflav', 'erdOne', 'github-actions', 'kckennylau'] kbuzzard
assignee:kbuzzard
1-39045
1 day ago
29-77992
29 days ago
29-78037
29 days
26790 FlAmmmmING
author:FlAmmmmING
feat(Combinatorics/Enumerative/Bell.lean): define standard Bell number --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-combinatorics 38/1 Mathlib/Combinatorics/Enumerative/Bell.lean 1 11 ['AntoineChambert-Loir', 'FlAmmmmING', 'eric-wieser', 'github-actions', 'kckennylau', 'madvorak'] awainverse
assignee:awainverse
1-39044
1 day ago
27-19723
27 days ago
27-19768
27 days
26793 FlAmmmmING
author:FlAmmmmING
feat(Algebra/Group /ForwardDiff.lean): add five theorems for forward difference --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import new-contributor t-algebra
label:t-algebra$
212/3 Mathlib/Algebra/Group/ForwardDiff.lean 1 35 ['AntoineChambert-Loir', 'DAE123456', 'FlAmmmmING', 'Ruben-VandeVelde', 'github-actions', 'kckennylau', 'madvorak'] mariainesdff
assignee:mariainesdff
1-39043
1 day ago
14-65633
14 days ago
27-18119
27 days
26835 Vtec234
author:Vtec234
feat(Tactic): dependent rewriting ct'd Add dependent rewrite tactics `rw!` and `rewrite!`. These operate by inserting casts in front of terms that would otherwise become type-incorrect after the rewrite. In the default mode, only proof terms are casted, so that (by proof irrelevance) no observable complexity is added. In the most liberal mode, the tactics never encounter the 'motive is not type correct' error, but may add casts that make the goal or other term very complex. Co-authored-by: Aaron Liu --- Continued from #23930. This has been discussed on Zulip [here](https://leanprover.zulipchat.com/#narrow/channel/239415-metaprogramming-.2F-tactics/topic/dependent.20rewrite.20tactic/with/504228516). See the included test file for example rewrites that this tactic can do. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta 935/0 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/DepRewrite.lean,MathlibTest/depRewrite.lean 4 6 ['Vtec234', 'github-actions', 'kmill', 'plp127'] eric-wieser
assignee:eric-wieser
1-39042
1 day ago
25-58161
25 days ago
25-58211
25 days
27109 pechersky
author:pechersky
feat(RingTheory/AdicValuation): valuation_surjective for both the base valuation and the one on the extension --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-analysis t-number-theory
label:t-algebra$
31/0 Mathlib/RingTheory/DedekindDomain/AdicValuation.lean,Mathlib/Topology/Algebra/Valued/ValuedField.lean 2 1 ['github-actions'] riccardobrasca
assignee:riccardobrasca
1-39041
1 day ago
18-62942
18 days ago
18-63023
18 days
27120 YaelDillies
author:YaelDillies
feat: the category of commutative bialgebras Define the bundled category `CommBialgCat R` of commutative bialgebras over a fixed commutative ring `R` along with the forgetful functor to `CommAlgCat`. From Toric Co-authored-by: Andrew Yang Co-authored-by: Michał Mrugała --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) toric t-algebra
label:t-algebra$
235/0 Mathlib.lean,Mathlib/Algebra/Category/CommBialgCat.lean 2 1 ['github-actions'] dagurtomas
assignee:dagurtomas
1-39039
1 day ago
18-53416
18 days ago
18-53486
18 days
27136 plp127
author:plp127
chore: mark argument explicit in `LinearOrder.toBiheytingAlgebra` Mark `α : Type*` explicit in `LinearOrder.toBiheytingAlgebra`. This matches better with what other similar reducible non-instances have. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order 17/14 Mathlib/Data/Fintype/Order.lean,Mathlib/Data/Nat/PartENat.lean,Mathlib/Order/CompleteLatticeIntervals.lean,Mathlib/Order/ConditionallyCompleteLattice/Basic.lean,Mathlib/Order/Fin/Basic.lean,Mathlib/Order/Heyting/Basic.lean 6 1 ['github-actions'] Vierkantor
assignee:Vierkantor
1-39038
1 day ago
18-22314
18 days ago
18-22309
18 days
27305 eric-wieser
author:eric-wieser
feat: instances for `ZeroHom` and `OneHom` This is motivated by wanting to write some lemmas about how the def in #27272 behaves on addition and scalar multiplcation, which requires these operations to first be defined. This shows that `ZeroHom` forms an `AddCommGroup` and `Module`, as well as analogous intermediate statements and `OneHom` results. --- - [x] depends on: #27318 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
188/8 Mathlib/Algebra/Group/Hom/Basic.lean,Mathlib/Algebra/Group/Hom/Instances.lean,Mathlib/Algebra/GroupWithZero/Action/Defs.lean,Mathlib/Algebra/GroupWithZero/Action/Hom.lean,Mathlib/Algebra/Module/Hom.lean,Mathlib/GroupTheory/GroupAction/DomAct/Basic.lean 6 3 ['eric-wieser', 'github-actions', 'mathlib4-dependent-issues-bot'] ericrbg
assignee:ericrbg
1-39037
1 day ago
9-3625
9 days ago
9-3608
9 days
27741 ShreckYe
author:ShreckYe
feat(Algebra/ModEq): add the `IsTrans` instance for `AddCommGroup.ModEq` The `trans` theorem is present for `AddCommGroup.ModEq` but there is no type class instance, while a similar instance is present for `Int.ModEq`, so I guess it should be missing. new-contributor t-algebra easy
label:t-algebra$
3/0 Mathlib/Algebra/ModEq.lean 1 2 ['ShreckYe', 'github-actions'] nobody
1-38877
1 day ago
1-38878
1 day ago
1-39251
1 day
27742 ChrisHughes24
author:ChrisHughes24
feat(Nat/nth): inequalities about Nat.nth --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data 58/0 Mathlib/Data/Nat/Nth.lean 1 1 ['github-actions'] nobody
1-38324
1 day ago
1-38332
1 day ago
1-38377
1 day
23181 YaelDillies
author:YaelDillies
refactor(Topology/UniformSpace): use `Rel` What's left in `UniformSpace.Defs` is precisely the theory of the uniformity filter. The motivation is that the theory of coverings and packings in both high dimensional probability and dynamics can be based on entourages, while they have little to do with the uniformity filter (indeed, entourages are in a sense a quantitative version of the uniformity filter). --- - [x] depends on: #25587 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology 787/600 Mathlib/Data/Rel.lean,Mathlib/Dynamics/TopologicalEntropy/CoverEntropy.lean,Mathlib/Dynamics/TopologicalEntropy/DynamicalEntourage.lean,Mathlib/Dynamics/TopologicalEntropy/NetEntropy.lean,Mathlib/Dynamics/TopologicalEntropy/Semiconj.lean,Mathlib/Dynamics/TopologicalEntropy/Subset.lean,Mathlib/InformationTheory/Hamming.lean,Mathlib/MeasureTheory/Measure/RegularityCompacts.lean,Mathlib/Topology/MetricSpace/BundledFun.lean,Mathlib/Topology/MetricSpace/PiNat.lean,Mathlib/Topology/Metrizable/Uniformity.lean,Mathlib/Topology/UniformSpace/Ascoli.lean,Mathlib/Topology/UniformSpace/Basic.lean,Mathlib/Topology/UniformSpace/Cauchy.lean,Mathlib/Topology/UniformSpace/Compact.lean,Mathlib/Topology/UniformSpace/CompactConvergence.lean,Mathlib/Topology/UniformSpace/Completion.lean,Mathlib/Topology/UniformSpace/Defs.lean,Mathlib/Topology/UniformSpace/DiscreteUniformity.lean,Mathlib/Topology/UniformSpace/Equicontinuity.lean,Mathlib/Topology/UniformSpace/HeineCantor.lean,Mathlib/Topology/UniformSpace/OfCompactT2.lean,Mathlib/Topology/UniformSpace/OfFun.lean,Mathlib/Topology/UniformSpace/Separation.lean,Mathlib/Topology/UniformSpace/Ultra/Basic.lean,Mathlib/Topology/UniformSpace/Ultra/Constructions.lean,Mathlib/Topology/UniformSpace/UniformApproximation.lean,Mathlib/Topology/UniformSpace/UniformConvergence.lean,Mathlib/Topology/UniformSpace/UniformEmbedding.lean 29 29 ['ADedecker', 'PatrickMassot', 'YaelDillies', 'b-mehta', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
1-36641
1 day ago
1-36665
1 day ago
64-43805
64 days
27716 kim-em
author:kim-em
chore: factor out lemmas from `LinearOrder ℚ` maintainer-merge t-algebra
label:t-algebra$
26/16 Mathlib/Algebra/Order/Ring/Unbundled/Rat.lean 1 3 ['github-actions', 'grunweg'] nobody
1-35363
1 day ago
1-35363
1 day ago
1-66220
1 day
25736 robin-carlier
author:robin-carlier
feat(AlgebraicTopology/SimplexCategory/GeneratorsRelations/NormalForms): Normal forms for `P_σ`s We prove that admissible lists indeed provide a normal form for morphisms of satisfying `P_σ`. To this end, we introduce `standardσ`, a construction that takes a list and turn it into a composition of `σ i`s in `SimplexCategoryGenRel`. We then prove that, thangs to the fifth simplicial identity, composition on the right corresponds to simplicial insertion in the list. This gives existence of a normal form for every morphism satisfying `P_σ`. For unicity, we introduce an auxiliary function `simplicialEvalσ : (List ℕ) → ℕ → ℕ` and show that for admissible lists, it lifts to `ℕ` the `orderHom` attached to `toSimplexCategory.map standardσ`, and that we can recover elements of the list only by looking at values of this function. Part of a series of PR formalising that `SimplexCategoryGenRel` is equivalent to `SimplexCategory`. --- - [x] depends on: #21744 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) --- *This PR continues the work from #21745.* *Original PR: https://github.com/leanprover-community/mathlib4/pull/21745* t-algebraic-topology large-import 253/7 Mathlib/AlgebraicTopology/SimplexCategory/GeneratorsRelations/NormalForms.lean 1 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
1-35108
1 day ago
1-35108
1 day ago
50-51271
50 days
26076 joelriou
author:joelriou
feat(AlgebraicTopology/SimplicialSet): uniqueness of the decomposition involving non-degenerate simplices Any simplex `x : X _⦋n⦌` of a simplicial set can be written in a unique way as `X.map f.op y` for an epimorphism `f : ⦋n⦌ ⟶ ⦋m⦌` and a non-degenerate `m`-simplex `y`. --- This PR continues the work from #21103. Original PR: https://github.com/leanprover-community/mathlib4/pull/21103 t-algebraic-topology 118/5 Mathlib/AlgebraicTopology/SimplexCategory/Basic.lean,Mathlib/AlgebraicTopology/SimplicialSet/Degenerate.lean 2 2 ['github-actions', 'joelriou'] nobody
1-35093
1 day ago
1-35093
1 day ago
44-44570
44 days
27166 joelriou
author:joelriou
feat(AlgebraicTopology): the functor `II : SimplexCategory ⥤ SimplexCategoryᵒᵖ` by Gabriel and Zisman In this file, we construct a cosimplicial object `SimplexCategory.II` in `SimplexCategoryᵒᵖ`, i.e. a functor `SimplexCategory ⥤ SimplexCategoryᵒᵖ`. If we identify `SimplexCategory` with the category of finite nonempty linearly ordered types, this functor could be interpreted as the contravariant functor which sends a finite nonempty linearly ordered type `T` to `T →o Fin 2`; in particular, it sends `Fin (n + 1)` to a linearly ordered type which is isomorphic to `Fin (n + 2)`. As a result, we define `SimplexCategory.II` as a functor which sends `⦋n⦌` to `⦋n + 1⦌`: on morphisms, it sends faces to degeneracies and vice versa. (I plan to use this in order to show that the topological realization from simplicial sets to `TopCat` preserves finite limits (at least after forgetting the topology), following the proof by Gabriel and Zisman.) --- Suggestions for a better (short) name are welcome. `II` is the name given is the original source. - [x] depends on: #27153 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebraic-topology 258/0 Mathlib.lean,Mathlib/AlgebraicTopology/SimplicialObject/II.lean 2 3 ['github-actions', 'joelriou', 'mathlib4-dependent-issues-bot'] nobody
1-34895
1 day ago
1-34895
1 day ago
16-52990
16 days
27090 TerenceGitH
author:TerenceGitH
feat(Topology, Archive/Examples): Kuratowski's closure-complement theorem (incl. sharpness) This is the outcome of a course project at Heidelberg University: https://matematiflo.github.io/CompAssistedMath2025/ feat(Topology): Kuratowski's closure-complement theorem "Topology/Kuratowski.lean" proves Kuratowski's closure-complement theorem, which says that if one repeatedly applies the closure and complement operators to a set in a topological space, at most 14 distinct sets can be obtained. feat(Archive/Examples): sharpness of Kuratowski's closure-complement theorem: "Examples/Kuratowski.lean" gives an example of a so-called "14-set" in ℝ, from which exactly 14 distinct sets can be obtained. Co-authored-by: Luis Sand @luiis-sd Co-authored-by: Leon Müller @leondieprobifi Co-authored-by: Junyan Xu @alreadydone --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-topology 386/0 Archive.lean,Archive/Examples/Kuratowski.lean,Mathlib.lean,Mathlib/Topology/Kuratowski.lean 4 8 ['alreadydone', 'github-actions', 'grunweg', 'wwylele'] j-loreaux
assignee:j-loreaux
1-33259
1 day ago
19-6087
19 days ago
19-7429
19 days
27552 Equilibris
author:Equilibris
chore: make typevec.arrow work over different universes This will be needed to allow `M.corec` to be generic across universes --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data new-contributor 16/10 Mathlib/Data/TypeVec.lean 1 3 ['Equilibris', 'github-actions', 'plp127'] nobody
1-32546
1 day ago
5-20357
5 days ago
5-20401
5 days
27309 kckennylau
author:kckennylau
feat(CategoryTheory): a presheaf on `CostructuredArrow F d` can be extended to a presheaf on `C` --- Zulip: [#Is there code for X? > over category via a functor](https://leanprover.zulipchat.com/#narrow/channel/217875-Is-there-code-for-X.3F/topic/over.20category.20via.20a.20functor/with/529574191) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory 218/0 Mathlib.lean,Mathlib/CategoryTheory/Comma/Presheaf/LeftExtension.lean 2 3 ['erdOne', 'github-actions', 'robin-carlier'] erdOne
assignee:erdOne
1-32296
1 day ago
12-22257
12 days ago
12-22307
12 days
25837 jt496
author:jt496
feat(Combinatorics/SimpleGraph): add homOfConnectedComponents and related results Given homomorphisms of each connected component of `G : SimpleGraph α` into `H : SimpleGraph β `give the corresponding `G →g H` Hence prove that G is n - colorable iff each connected component is n - colorable. Also prove that G is 2-colorable iff it does not contain an odd length loop (closed walk). I wasn't sure where to put this - it probably belongs in SimpleGraph.ConcreteColorings? --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) --- *This PR continues the work from #24546.* *Original PR: https://github.com/leanprover-community/mathlib4/pull/24546* t-combinatorics 36/0 Mathlib/Combinatorics/SimpleGraph/Coloring.lean,Mathlib/Combinatorics/SimpleGraph/ConcreteColorings.lean,Mathlib/Combinatorics/SimpleGraph/Connectivity/Connected.lean 3 6 ['b-mehta', 'github-actions'] b-mehta
assignee:b-mehta
1-31094
1 day ago
49-43900
1 month ago
49-43883
49 days
25952 101damnations
author:101damnations
feat(RepresentationTheory/Homological/GroupHomology/Functoriality): the degree 1 part of the corestriction-coinflation exact sequence when the subgroup acts trivially Given a normal subgroup `S` of `G` and a `G`-representation `A` on which `S` acts trivially, this PR defines the short complex `H₁(S, A) ⟶ H₁(G, A) ⟶ H₁(G ⧸ S, A)` induced by the natural inclusion `S → G` and projection `G → G / S`. We show it is exact and that the righthand map is an epimorphism. --- - [x] depends on: #21652 - [x] depends on: #21732 - [x] depends on: #21733 - [x] depends on: #21735 - [x] depends on: #21736 - [x] depends on: #21738 - [x] depends on: #25868 - [x] depends on: #25873 - [x] depends on: #25880 - [x] depends on: #25884 - [x] depends on: #25888 - [x] depends on: #25939 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) --- *Earlier version at #22654* maintainer-merge t-algebra
label:t-algebra$
142/2 Mathlib/RepresentationTheory/Homological/GroupCohomology/Functoriality.lean,Mathlib/RepresentationTheory/Homological/GroupHomology/Functoriality.lean 2 n/a ['101damnations', 'github-actions', 'kbuzzard', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
1-30828
1 day ago
unknown
unknown
25966 b-reinke
author:b-reinke
feat(GroupTheory/FreeGroup): add predicate for reduced words This PR adds the predicate of reduced words `IsReduced` in the construction of free groups. It is shown that `reduce` and `toWord` produce reduced words. This is done in preparation for the theory of cyclically reduced words. Upstreamed from the [EquationalTheories](https://github.com/teorth/equational_theories) project. --- This PR continues the work from #23368. Original PR: https://github.com/leanprover-community/mathlib4/pull/23368 maintainer-merge t-algebra
label:t-algebra$
82/0 Mathlib/GroupTheory/FreeGroup/Basic.lean,Mathlib/GroupTheory/FreeGroup/Reduce.lean 2 35 ['YaelDillies', 'b-reinke', 'github-actions', 'vlad902'] nobody
1-27886
1 day ago
1-38347
1 day ago
45-29201
45 days
27270 EtienneC30
author:EtienneC30
chore: turn WithLp into a structure Turn `WithLp` into a one field structure, as was suggested many times on Zulip and discussed here: https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/defeq.20abuse.20in.20.60WithLp.60/near/526234806. Here is what this PR does: - The instances on `WithLp p α` which were defeq to those on `α` (algebraic instances, topology, uniformity, bornology) are now pulled back from `α` along `WithLp.equiv p α`. A few declarations are added to ease the process, such as versions of `WithLp.equiv` as a homeomorphism or a uniform isomorphism. - It introduces some definitions to equip `α × β` with the Lp distance, and similarly for `Π i, α i`. This is then used to define relevant instances on type synonyms, such as for matrix norms. - The PR fixes all the defeq abuses (which break obviously). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-analysis 756/399 Archive/Hairer.lean,Mathlib.lean,Mathlib/Algebra/Module/ZLattice/Covolume.lean,Mathlib/Analysis/Analytic/WithLp.lean,Mathlib/Analysis/CStarAlgebra/Matrix.lean,Mathlib/Analysis/Calculus/ContDiff/WithLp.lean,Mathlib/Analysis/Calculus/FDeriv/WithLp.lean,Mathlib/Analysis/InnerProductSpace/PiL2.lean,Mathlib/Analysis/InnerProductSpace/ProdL2.lean,Mathlib/Analysis/InnerProductSpace/Spectrum.lean,Mathlib/Analysis/Matrix.lean,Mathlib/Analysis/Normed/Algebra/TrivSqZeroExt.lean,Mathlib/Analysis/Normed/Algebra/UnitizationL1.lean,Mathlib/Analysis/Normed/Lp/LpEquiv.lean,Mathlib/Analysis/Normed/Lp/MeasurableSpace.lean,Mathlib/Analysis/Normed/Lp/PiLp.lean,Mathlib/Analysis/Normed/Lp/ProdLp.lean,Mathlib/Analysis/Normed/Lp/WithLp.lean,Mathlib/Analysis/Quaternion.lean,Mathlib/Analysis/RCLike/Inner.lean,Mathlib/Analysis/SpecialFunctions/Gaussian/FourierTransform.lean,Mathlib/Combinatorics/Additive/AP/Three/Behrend.lean,Mathlib/Geometry/Manifold/Instances/Icc.lean,Mathlib/Geometry/Manifold/Instances/Real.lean,Mathlib/LinearAlgebra/Matrix/PosDef.lean,Mathlib/LinearAlgebra/Matrix/Spectrum.lean,Mathlib/MeasureTheory/Measure/Haar/InnerProductSpace.lean,Mathlib/MeasureTheory/Measure/Haar/OfBasis.lean,Mathlib/MeasureTheory/Measure/Lebesgue/VolumeOfBalls.lean,Mathlib/NumberTheory/NumberField/CanonicalEmbedding/Basic.lean,Mathlib/NumberTheory/NumberField/Ideal/Asymptotics.lean 31 5 ['eric-wieser', 'github-actions', 'leanprover-community-bot-assistant'] nobody
1-27369
1 day ago
1-32479
1 day ago
13-70322
13 days
27751 Vierkantor
author:Vierkantor
feat: `erw?` supports all arguments that `erw` does This PR teaches `erw?` how to deal with multiple arguments and how to rewrite at a hypothesis, so that it can be used everywhere that `erw` can. (And ideally `erw` can then be removed from those places.) In addition to the new tests, I picked a few places in the library to run as test cases with more complicated terms (but `extract_goals` didn't really work there...) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta 146/15 Mathlib/Tactic/ErwQuestion.lean,MathlibTest/ErwQuestion.lean 2 1 ['github-actions'] nobody
1-26441
1 day ago
1-26520
1 day ago
1-26503
1 day
27419 grunweg
author:grunweg
chore(IntegrableOn): generalise one more section to enorms --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) carleson maintainer-merge t-measure-probability 139/96 Mathlib/Analysis/MellinTransform.lean,Mathlib/Analysis/SpecialFunctions/ImproperIntegrals.lean,Mathlib/Analysis/SpecialFunctions/Integrability/Basic.lean,Mathlib/Analysis/SpecialFunctions/Integrals/LogTrigonometric.lean,Mathlib/MeasureTheory/Integral/ExpDecay.lean,Mathlib/MeasureTheory/Integral/IntegrableOn.lean,Mathlib/MeasureTheory/Integral/IntervalIntegral/Basic.lean,Mathlib/MeasureTheory/Integral/IntervalIntegral/FundThmCalculus.lean,Mathlib/MeasureTheory/Integral/IntervalIntegral/Periodic.lean,Mathlib/MeasureTheory/Measure/Lebesgue/Integral.lean,Mathlib/NumberTheory/AbelSummation.lean,Mathlib/NumberTheory/LSeries/SumCoeff.lean 12 8 ['YaelDillies', 'github-actions', 'grunweg', 'sgouezel'] YaelDillies
assignee:YaelDillies
1-25124
1 day ago
1-25124
1 day ago
8-49359
8 days
27754 Parcly-Taxel
author:Parcly-Taxel
feat: `finCycle` as iterated `finRotate` Originally used in #25786, but eventually discovered to be unnecessary. t-logic 26/5 Mathlib/Logic/Equiv/Fin/Rotate.lean 1 1 ['github-actions'] nobody
1-22663
1 day ago
1-22668
1 day ago
1-22721
1 day
25786 Parcly-Taxel
author:Parcly-Taxel
feat: IMO 2001 Q4 IMO maintainer-merge 106/0 Archive.lean,Archive/Imo/Imo2001Q4.lean 2 11 ['Parcly-Taxel', 'dwrensha', 'github-actions', 'leanprover-community-bot-assistant'] dwrensha
assignee:dwrensha
1-22146
1 day ago
1-22146
1 day ago
48-53017
48 days
27757 mbkybky
author:mbkybky
feat(RingTheory): `IsTensorProduct` versions of the lemmas about tensoring with a flat module preserves injections Add some lemmas about `IsTensorProduct` and the `IsTensorProduct` versions of the lemmas about tensoring with a flat module preserves injections. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
220/19 Mathlib/RingTheory/Flat/Basic.lean,Mathlib/RingTheory/IsTensorProduct.lean 2 1 ['github-actions'] nobody
1-21418
1 day ago
1-21606
1 day ago
1-21657
1 day
27691 bryangingechen
author:bryangingechen
ci: rebuild until `lake build --no-build` succeeds This should hopefully help with the CI failing in the cache verification step in the Post-Build job, as recently observed on various PRs in: [#mathlib4 > Failing CI @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Failing.20CI/near/530878203). Also adds `-v` to the `lake build --no-build` steps as well as `-wfail` to the `Archive` and `Counterexamples` build steps (cf. #19633 for the latter). The log output will be long, so we use [GitHub's log grouping feature](https://docs.github.com/en/actions/reference/workflows-and-actions/workflow-commands#grouping-log-lines) to make the logs easier to navigate. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) CI 143/36 .github/build.in.yml,.github/workflows/bors.yml,.github/workflows/build.yml,.github/workflows/build_fork.yml,scripts/README.md,scripts/lake-build-with-retry.sh 6 10 ['bryangingechen', 'github-actions', 'grunweg', 'kim-em', 'tydeu'] nobody
1-18335
1 day ago
1-22967
1 day ago
1-58003
1 day
26464 joelriou
author:joelriou
feat(LinearAlgebra): generators of pi tensor products In this PR, we show that the `R`-module `⨂[R] i, M i` is finitely generated if the index type is finite and all `M i` are finitely generated. This follows from a more precise result about generators of `⨂[R] i, M i`. --- This PR continues the work from #18725. Original PR: https://github.com/leanprover-community/mathlib4/pull/18725 file-removed t-algebra
label:t-algebra$
268/4 Mathlib.lean,Mathlib/Analysis/NormedSpace/PiTensorProduct/ProjectiveSeminorm.lean,Mathlib/Data/SubtypeNeLift.lean,Mathlib/LinearAlgebra/PiTensorProduct/Basic.lean,Mathlib/LinearAlgebra/PiTensorProduct/Finite.lean,Mathlib/LinearAlgebra/PiTensorProduct/Generators.lean,Mathlib/LinearAlgebra/TensorPower/Basic.lean,Mathlib/RingTheory/PiTensorProduct.lean,Mathlib/SetTheory/Cardinal/Finite.lean 9 13 ['eric-wieser', 'github-actions', 'joelriou', 'leanprover-community-bot-assistant'] nobody
1-17796
1 day ago
1-26234
1 day ago
31-51756
31 days
27762 plp127
author:plp127
chore(AbstractCompletion): universe polymorphism --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology 17/16 Mathlib/Topology/UniformSpace/AbstractCompletion.lean 1 1 ['github-actions'] nobody
1-16472
1 day ago
1-16542
1 day ago
1-16590
1 day
25089 Bergschaf
author:Bergschaf
feat(Order/Sublocale): definition of sublocales There are several possible definition of sublocales. I used one from [nlab](https://ncatlab.org/nlab/show/sublocale) which states that a sublocale is a subset of a locale which is closed under all meets and for any `s ∈ S` and `x ∈ X`, we have `(x ⇨ s) ∈ S`. This PR also includes an order isomorphism between `(Nucleus)ᵒᵈ` and `Sublocale`. --- I am open to better name suggestions for the order isomorphism. - [x] depends on: #24941 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) maintainer-merge t-order 327/30 Mathlib.lean,Mathlib/Order/Hom/Lattice.lean,Mathlib/Order/Nucleus.lean,Mathlib/Order/Sublocale.lean,Mathlib/Order/Synonym.lean,docs/references.bib 6 91 ['Bergschaf', 'YaelDillies', 'b-mehta', 'bryangingechen', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'xhalo32'] bryangingechen
assignee:bryangingechen
1-15916
1 day ago
55-6532
1 month ago
68-72352
68 days
27763 j-loreaux
author:j-loreaux
feat: define morphism type `StarMonoidHom` This defines star-preserving monoid homomorphisms between star monoids. The primary motivation for these morphisms is to provide a target type for morphisms which induce a corresponding morphism between the unitary groups in a star monoid. Without this type, there is no concrete type for [unitary.map](https://leanprover-community.github.io/mathlib4_docs/Mathlib/Algebra/Star/Unitary.html#unitary.map) and we end up resorting to morphisms *classes* instead, which is suboptimal. See [Zulip](https://leanprover.zulipchat.com/#narrow/channel/113489-new-members/topic/.E2.9C.94.20Golfing.20matrix.20group.20coercion/near/528000462) for the problem which motivated the creation of this type. --- In a follow-up PR, I will redefine `unitary.map` so that it takes a `StarMonoidHom` as an argument and also outputs a `StarMonoidHom`. I will also add `unitary.mapEquiv` for a version which does the same for `StarMulEquiv`. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
335/0 Mathlib.lean,Mathlib/Algebra/Star/MonoidHom.lean 2 1 ['github-actions'] nobody
1-14653
1 day ago
1-14690
1 day ago
1-14703
1 day
27696 pechersky
author:pechersky
feat(Padic/WithVal): WithVal v is isomorphic to Q_p as fields and uniform spaces On the way to a topological ring equiv --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-number-theory
label:t-algebra$
187/0 Mathlib.lean,Mathlib/NumberTheory/Padics/PadicNumbers.lean,Mathlib/NumberTheory/Padics/WithVal.lean 3 1 ['github-actions'] nobody
1-12040
1 day ago
2-7970
2 days ago
2-7967
2 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/) t-set-theory 58/16 Mathlib/SetTheory/ZFC/Basic.lean,Mathlib/SetTheory/ZFC/Ordinal.lean 2 3 ['b-mehta', 'github-actions', 'vihdzp'] nobody
1-8414
1 day ago
1-77206
1 day ago
1-77250
1 day
27786 staroperator
author:staroperator
feat(GroupTheory/Finiteness): `AddMonoid.FG ℕ` and `AddGroup.FG ℤ` Note: [`Module.Finite.self`](https://leanprover-community.github.io/mathlib4_docs/Mathlib/RingTheory/Finiteness/Basic.html#Module.Finite.self) gives equivalent results as `Module.Finite ℕ ℕ` and `Module.Finite ℤ ℤ`. But there is no instance from `Module.Finite` to `AddMonoid.FG` (there is one converse, [AddMonoid.FG.to_moduleFinite_nat](https://leanprover-community.github.io/mathlib4_docs/Mathlib/RingTheory/Finiteness/Defs.html#AddMonoid.FG.to_moduleFinite_nat)). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
10/0 Mathlib/GroupTheory/Finiteness.lean 1 1 ['github-actions'] nobody
1-6254
1 day ago
1-6261
1 day ago
1-6307
1 day
27787 staroperator
author:staroperator
feat(GroupTheory/Finiteness): instance `Monoid.fg_of_group_fg` This makes one direction of `Group.fg_iff_monoid_fg` an instance. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
5/0 Mathlib/GroupTheory/Finiteness.lean 1 1 ['github-actions'] nobody
1-6152
1 day ago
1-6158
1 day ago
1-6204
1 day
27449 kckennylau
author:kckennylau
feat(Topology): finite dimensional vector space over locally compact complete space is locally compact *From the 2025 Local Class Field Theory Workshop.* --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) maintainer-merge t-topology 18/0 Mathlib/Topology/Algebra/Module/FiniteDimension.lean 1 7 ['ADedecker', 'github-actions', 'kbuzzard', 'kckennylau', 'mariainesdff'] nobody
1-5898
1 day ago
4-22373
4 days ago
4-57131
4 days
27511 Nebula691
author:Nebula691
feat(Algebra/QuadraticAlgebra) : Define Quadratic Algebra co-authored-by : Edison Xie co-authored-by : Kenny Lau --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra
label:t-algebra$
418/0 Mathlib.lean,Mathlib/Algebra/QuadraticAlgebra.lean 2 59 ['Whysoserioushah', 'eric-wieser', 'github-actions', 'kckennylau'] nobody
1-5484
1 day ago
6-22221
6 days ago
6-22265
6 days
27094 smorel394
author:smorel394
feat(Algebra.Category.FGModuleCat.Colimits): the category of finitely generated modules has finite colimits Prove that the forgetful functor from `FGModuleCat k` to `ModuleCat k` creates finite colimits, and hence that `FGModuleCat k` has finite colimits. - [ ] depends on: #27092 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
70/0 Mathlib.lean,Mathlib/Algebra/Category/FGModuleCat/Colimits.lean 2 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
1-4754
1 day ago
2-9797
2 days ago
2-10975
2 days
27788 grunweg
author:grunweg
chore(Topology/Algebra/Support): misc. clean-ups; rename `HasCompactSupport.inv'` to `inv` Companion to #27777. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology 29/23 Mathlib/Analysis/Convolution.lean,Mathlib/Topology/Algebra/Support.lean,Mathlib/Topology/ContinuousMap/BoundedCompactlySupported.lean 3 2 ['github-actions', 'grunweg'] nobody
1-2302
1 day ago
1-2302
1 day ago
1-2307
1 day
9915 eric-wieser
author:eric-wieser
refactor: Add norm_num machinery for NNRat This splits the previous `isRat` primitive into `isNNRat` and `isNegNNRat`, where only the latter carries around a `DivisionRing` instance. This means that `norm_num` works on `NNReal` and `NNRat`. Co-authored-by: Aaron Liu --- - [x] depends on: #9951 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-meta
label:t-algebra$
758/237 Mathlib/Analysis/SpecialFunctions/Log/Basic.lean,Mathlib/Analysis/SpecialFunctions/Pow/Real.lean,Mathlib/Data/Rat/Floor.lean,Mathlib/Tactic/NormNum/Basic.lean,Mathlib/Tactic/NormNum/BigOperators.lean,Mathlib/Tactic/NormNum/Eq.lean,Mathlib/Tactic/NormNum/Ineq.lean,Mathlib/Tactic/NormNum/Inv.lean,Mathlib/Tactic/NormNum/Irrational.lean,Mathlib/Tactic/NormNum/OfScientific.lean,Mathlib/Tactic/NormNum/Pow.lean,Mathlib/Tactic/NormNum/RealSqrt.lean,Mathlib/Tactic/NormNum/Result.lean,Mathlib/Tactic/Positivity/Core.lean,Mathlib/Tactic/Ring/Basic.lean,Mathlib/Tactic/Ring/RingNF.lean,MathlibTest/norm_num.lean,MathlibTest/norm_num_ext.lean,MathlibTest/ring.lean,scripts/nolints.json 20 8 ['eric-wieser', 'github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'plp127'] kim-em
assignee:kim-em
1-2143
1 day ago
19-17410
19 days ago
29-16795
29 days
19668 YaelDillies
author:YaelDillies
refactor: define `≤`/`<` on `WithBot`/`WithTop` by induction The motivation for this change is that it is really confusing to run `intro r s shouldnthaveintroedthat` on a goal of the form `∀ r s : ℝ≥0∞, r ≤ s` and get the nonsense-looking goal `r = ↑shouldnthaveintroedthat → ∃ b : α, s = ↑b ∧ shouldnthaveintroedthat ≤ b⟩` instead of an error, and similarly when destructing something of the form `∃ r s : ℝ≥0∞, r < s`. Furthermore, I suspect this improves performance. --- - [x] depends on: #20317 - [x] depends on: #20318 - [x] depends on: #21274 - [x] depends on: #22109 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order 68/51 Mathlib/Algebra/Order/Monoid/Unbundled/WithTop.lean,Mathlib/Analysis/Analytic/OfScalars.lean,Mathlib/Analysis/Oscillation.lean,Mathlib/Data/Finset/Lattice/Fold.lean,Mathlib/Data/Finset/Max.lean,Mathlib/LinearAlgebra/Eigenspace/Triangularizable.lean,Mathlib/MeasureTheory/Integral/Lebesgue/Countable.lean,Mathlib/MeasureTheory/Measure/LevyProkhorovMetric.lean,Mathlib/Order/Interval/Basic.lean,Mathlib/Order/Interval/Set/WithBotTop.lean,Mathlib/Order/KrullDimension.lean,Mathlib/Order/WithBot.lean,Mathlib/Probability/Moments/Variance.lean,Mathlib/RingTheory/PowerBasis.lean,Mathlib/Topology/MetricSpace/Holder.lean,Mathlib/Topology/MetricSpace/HolderNorm.lean,MathlibTest/hint.lean 17 20 ['YaelDillies', 'b-mehta', 'eric-wieser', 'github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'urkud'] Vierkantor
assignee:Vierkantor
1-2142
1 day ago
76-49900
2 months ago
126-42450
126 days
24528 chrisflav
author:chrisflav
feat(AlgebraicGeometry): directed covers Directed covers are covers, where every intersection can be covered by a component of the cover. For open covers this is equivalent to the images forming a basis of the topology. If a cover is directed, the compatibility conditions for gluing become easier, because only compatibility with the transition maps needs to be checked. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebraic-geometry 233/0 Mathlib.lean,Mathlib/AlgebraicGeometry/Cover/Directed.lean 2 6 ['chrisflav', 'erdOne', 'github-actions', 'joelriou', 'leanprover-community-bot-assistant'] mattrobball
assignee:mattrobball
1-2141
1 day ago
70-31189
2 months ago
87-16209
87 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/) new-contributor t-combinatorics 16/0 Mathlib/Combinatorics/SimpleGraph/Trails.lean 1 3 ['IvanRenison', 'github-actions'] kmill
assignee:kmill
1-2140
1 day ago
66-80091
2 months ago
66-80144
66 days
25795 dagurtomas
author:dagurtomas
chore(Condensed): introduce an abbrev for the equivalence of light condensed sets with a category of sheaves on a small site --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) --- *This PR continues the work from #24522.* *Original PR: https://github.com/leanprover-community/mathlib4/pull/24522* t-condensed 39/0 Mathlib.lean,Mathlib/Condensed/Light/Small.lean 2 1 ['github-actions'] joneugster
assignee:joneugster
1-2137
1 day ago
50-39546
1 month ago
50-39528
50 days
25856 MichaelStollBayreuth
author:MichaelStollBayreuth
perf(Data.Real.Sqrt): make Real.sqrt irreducible We try to see what happens if we make Real.sqrt irreducible. There are cases where this makes unification very significantly faster, compare [#mathlib4 > Coercion triggers timeout @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Coercion.20triggers.20timeout/near/517177117). (Migrated manually from #24752) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) migrated-from-branch t-data 1/0 Mathlib/Data/Real/Sqrt.lean 1 1 ['github-actions'] ericrbg
assignee:ericrbg
1-2136
1 day ago
48-32701
1 month ago
48-36404
48 days
26287 mbkybky
author:mbkybky
feat(Data/ENat/Lattice): coercion to `WithBot ℕ∞` commutes with `biSup` The coercion from `ℕ∞` to `WithBot ℕ∞` commutes with `biSup` and `biInf`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data 19/0 Mathlib/Data/ENat/Lattice.lean 1 1 ['github-actions'] ericrbg
assignee:ericrbg
1-2136
1 day ago
39-61420
1 month ago
39-69169
39 days
26347 mans0954
author:mans0954
feature(Data/Finset/RangeDistance): abs_sub_lt_of_mem_finset_range This PR continues the work from #23161. Original PR: https://github.com/leanprover-community/mathlib4/pull/23161 30/0 Mathlib.lean,Mathlib/Algebra/Order/Group/Unbundled/Abs.lean,Mathlib/Data/Finset/RangeDistance.lean 3 2 ['github-actions', 'mans0954'] alreadydone
assignee:alreadydone
1-2135
1 day ago
38-50730
1 month ago
38-50711
38 days
26370 b-mehta
author:b-mehta
chore(Archive): golf and generalise ascending-descending sequences This proof was 5 years old, not in a good generality, and overly long. We fix the latter two points. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data 96/120 Archive/Wiedijk100Theorems/AscendingDescendingSequences.lean 1 12 ['b-mehta', 'github-actions', 'grunweg'] ericrbg
assignee:ericrbg
1-2132
1 day ago
36-40680
1 month ago
38-9217
38 days
26489 chrisflav
author:chrisflav
refactor(RingTheory/RingHom): factor out proofs for `Algebra.FinitePresentation` The current way to use locality of a given property of algebras is to convert everything into the language of `RingHom`s and then for example the `RingHom.OfLocalizationSpanTarget` API. This has two disadvantages: 1. The ring hom property API fixes the universes of source and target to be the same, hence we unnecessarily lose out on some universe generality. 2. The results for `RingHom`s are proven by translating everything in terms of `Algebra`, so we duplicate the translation steps. This PR refactors `RingHom.FinitePresentation` to do all locality proofs in the language of `Algebra`s and translate it into the corresponding `RingHom.OfLocalizationSpan{Target}` in the last step. We also streamline some of the translation proofs by unifying the API. --- - [x] depends on: #22931 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) This PR continues the work from #22930. Original PR: https://github.com/leanprover-community/mathlib4/pull/22930 t-algebra
label:t-algebra$
62/77 Mathlib/RingTheory/RingHom/FinitePresentation.lean 1 4 ['chrisflav', 'erdOne', 'github-actions', 'mathlib4-dependent-issues-bot'] kim-em
assignee:kim-em
1-2131
1 day ago
34-28681
1 month ago
34-28727
34 days
26811 loefflerd
author:loefflerd
feat(LinearAlgebra/Projectivization): GL(V) action Some API around projective spaces and general linear groups: - an equiv between V and W gives an equiv between GL(V) and GL(W) - GL(V) acts on the projectivization of V - GL 2 K acts on `OnePoint K` (which is the projectivization of `K x K`) I am adding these because I need them to define cusps in modular form theory, but they are hopefully something of general usefulness beyond that. --- - [x] depends on: #27104 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-algebra
label:t-algebra$
146/3 Mathlib.lean,Mathlib/LinearAlgebra/GeneralLinearGroup.lean,Mathlib/LinearAlgebra/Projectivization/GLAction.lean,Mathlib/Topology/Compactification/OnePoint/ProjectiveLine.lean 4 26 ['bjoernkjoshanssen', 'eric-wieser', 'github-actions', 'loefflerd', 'mathlib4-dependent-issues-bot'] adomani
assignee:adomani
1-2131
1 day ago
17-45091
17 days ago
25-81383
25 days
26909 gasparattila
author:gasparattila
feat(LinearAlgebra/Projectivization/Subspace): correspondence between linear and projective subspaces --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra
label:t-algebra$
51/3 Mathlib/LinearAlgebra/Projectivization/Subspace.lean 1 1 ['github-actions'] Vierkantor
assignee:Vierkantor
1-2130
1 day ago
24-5522
24 days ago
24-5570
24 days
27184 JovanGerb
author:JovanGerb
chore(Order/Filter/Basic): write lemmas in point-free style This PR writes the congruence lemmas about filtered equality and about asymptotic equivalence in a point-free style. This is so that they can then be tagged with `@[gcongr]`. Some of the old versions have been kept with a `fun_` name. And apparently the import size has decreased as a bonus :) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order 43/28 Mathlib/Analysis/Asymptotics/AsymptoticEquivalent.lean,Mathlib/Analysis/Normed/Ring/Units.lean,Mathlib/MeasureTheory/Function/LpSpace/Basic.lean,Mathlib/MeasureTheory/Function/LpSpace/Indicator.lean,Mathlib/MeasureTheory/Integral/Lebesgue/Add.lean,Mathlib/Order/Filter/Basic.lean,Mathlib/Order/Filter/Map.lean,Mathlib/Probability/Density.lean 8 4 ['JovanGerb', 'eric-wieser', 'github-actions'] bryangingechen
assignee:bryangingechen
1-2128
1 day ago
16-81564
16 days ago
16-81608
16 days
27355 alreadydone
author:alreadydone
feat(Algebra): annihilator of fg module over PID is ann of some element Live coding at *Formalizing Class Field Theory* for the finite case of the normal basis theorem --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
50/0 Mathlib/Algebra/Module/PID.lean,Mathlib/RingTheory/Ideal/Maps.lean 2 6 ['alreadydone', 'github-actions', 'kckennylau'] jcommelin
assignee:jcommelin
1-2125
1 day ago
10-13151
10 days ago
10-13134
10 days
27715 dupuisf
author:dupuisf
feat(CStarAlgebra): `a => a ^ p` is operator monotone for `p ∈ Icc 0 1` This PR shows that `a => a ^ p` is operator monotone for `p ∈ Icc 0 1`, i.e. that `CFC.nnrpow`, `CFC.rpow` and `CFC.sqrt` are monotone, using the integral representation for the power function. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-analysis 307/12 Mathlib/Algebra/Algebra/Spectrum/Quasispectrum.lean,Mathlib/Analysis/Normed/Algebra/Spectrum.lean,Mathlib/Analysis/SpecialFunctions/ContinuousFunctionalCalculus/Rpow/IntegralRepresentation.lean,Mathlib/Topology/ContinuousOn.lean 4 1 ['github-actions'] nobody
1-611
1 day ago
1-616
1 day ago
1-599
1 day
25453 JovanGerb
author:JovanGerb
perf(Algebra/Homology/HomotopyCategory): use explicit universe parameter in `Category` As we have seen before, writing `Category.{v}` instead of `Category` avoids a nasty universe level metavariable, and this helps to speed up unification. The changes in this PR are somewhat arbitrary, but it serves as an example for this principle. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
9/6 Mathlib/Algebra/Homology/HomotopyCategory/DegreewiseSplit.lean,Mathlib/Algebra/Homology/HomotopyCategory/MappingCone.lean,Mathlib/Algebra/Homology/HomotopyCategory/Triangulated.lean 3 5 ['JovanGerb', 'github-actions', 'leanprover-bot'] chrisflav
assignee:chrisflav
0-83973
23 hours ago
58-5950
1 month ago
58-6000
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 t-meta 75/3 Mathlib/Util/Delaborators.lean,Mathlib/Util/PPOptions.lean,MathlibTest/delaborators.lean 3 11 ['JovanGerb', 'Rob23oba', 'eric-wieser', 'github-actions'] alexjbest
assignee:alexjbest
0-83972
23 hours ago
57-2481
1 month ago
57-2538
57 days
25970 wwylele
author:wwylele
feat(RingTheory): decompose archimedean classes of HahnSeries In preparation for #25140, this connects archimedean class and HahnSeries --- - [x] depends on: #26773 - [x] depends on: #26787 - [x] depends on: #26788 - [x] depends on: #26789 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import 357/2 Mathlib/Algebra/Order/Archimedean/Class.lean,Mathlib/RingTheory/HahnSeries/Lex.lean 2 14 ['ScottCarnahan', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'wwylele'] alreadydone
assignee:alreadydone
0-83971
23 hours ago
20-74585
20 days ago
39-20778
39 days
26189 tb65536
author:tb65536
feat(FieldTheory/Galois/Basic): Add simp-lemma for `FixedPoints.intermediateField` This PR adds a simp-lemma `FixedPoints.mem_intermediateField_iff` for the definition `FixedPoints.intermediateField`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
4/0 Mathlib/FieldTheory/Galois/Basic.lean 1 1 ['github-actions'] joneugster
assignee:joneugster
0-83970
23 hours ago
39-22370
1 month ago
42-80019
42 days
26192 kckennylau
author:kckennylau
feat(LinearAlgebra): symmetric tensor power --- Zulip: [#mathlib4 > Proposal: Symmetric Tensor Power](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Proposal.3A.20Symmetric.20Tensor.20Power/with/524795235) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
129/0 Mathlib.lean,Mathlib/LinearAlgebra/TensorPower/Symmetric.lean 2 6 ['AntoineChambert-Loir', 'erdOne', 'eric-wieser', 'github-actions', 'kckennylau'] mattrobball
assignee:mattrobball
0-83969
23 hours ago
42-78001
1 month ago
42-78044
42 days
26201 scholzhannah
author:scholzhannah
feat: subcomplexes of a classical CW complex This PR defines subcomplexes of a (classical relative) CW complex to be a closed subspace which is a union of open cells. It provides additional definitions for alternative ways to describe subcomplexes. Lastly, it refactors the definition of the skeleton to define it as a subcomplex. Co-authored-by: Floris van Doorn --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology 213/25 Mathlib/Topology/CWComplex/Classical/Basic.lean 1 2 ['github-actions', 'leanprover-community-bot-assistant'] ADedecker
assignee:ADedecker
0-83968
23 hours ago
21-32218
21 days ago
40-57557
40 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/) new-contributor t-analysis 365/0 Mathlib.lean,Mathlib/Analysis/Calculus/FDeriv/Partial.lean,Mathlib/Analysis/Normed/Operator/BoundedLinearMaps.lean 3 7 ['YaelDillies', 'agjftucker', 'github-actions', 'igorkhavkine', 'mathlib4-dependent-issues-bot'] sgouezel
assignee:sgouezel
0-83967
23 hours ago
36-48730
1 month ago
37-34467
37 days
26841 xroblot
author:xroblot
feat(FieldTheory/IsGalois): map induced by the restriction to a subfield For `E/L` a field extension and `K` a subfield of `E`, we define the map `(E ≃ₐ[L] E) →* (K ≃ₐ[F] K)` induced by the restriction to `K` (with `F` a subfield of `K` and `L` such that `K/F` is normal) and study when it is injective and surjective. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
63/0 Mathlib/FieldTheory/Galois/Basic.lean 1 1 ['github-actions'] Vierkantor
assignee:Vierkantor
0-83964
23 hours ago
25-49248
25 days ago
25-49294
25 days
27066 vasnesterov
author:vasnesterov
feat(Tactic/Order): frontend for `order` * Support `order [h1, h2]` and `order only [h1, h2]` syntax. * Split conjunctions while extracting facts from the context. E.g. hypotheses in the form `A ∧ B` are converted into two facts `A` and `B`. * Similarly, extract facts from existential quantifiers in the hypotheses. --- - [x] depends on: #26354 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) This PR continues the work from #22073. Original PR: https://github.com/leanprover-community/mathlib4/pull/22073 t-meta 91/37 Mathlib.lean,Mathlib/Tactic/Linarith/Frontend.lean,Mathlib/Tactic/Order.lean,Mathlib/Tactic/Order/CollectFacts.lean,Mathlib/Util/ElabWithoutMVars.lean,MathlibTest/order.lean 6 22 ['JovanGerb', 'github-actions', 'mathlib4-dependent-issues-bot', 'vasnesterov'] alexjbest
assignee:alexjbest
0-83960
23 hours ago
19-43887
19 days ago
19-43915
19 days
27304 jano-wol
author:jano-wol
feat: invariant dual submodules define Lie ideals Invariant dual submodules define Lie ideals --- PR shows that Invariant dual submodules define Lie ideals. This work is part of the framework: https://github.com/orgs/leanprover-community/projects/17 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
358/0 Mathlib.lean,Mathlib/Algebra/Lie/Weights/InvariantSubmoduleLieIdeal.lean,Mathlib/Algebra/Lie/Weights/Killing.lean,Mathlib/Algebra/Lie/Weights/RootSystem.lean 4 1 ['github-actions'] jcommelin
assignee:jcommelin
0-83958
23 hours ago
12-35497
12 days ago
12-35543
12 days
27380 chrisflav
author:chrisflav
feat(Category/Ring): `Algebra.IsPushout` iff `CategoryTheory.IsPushout` In particular, `RingHom.IsStableUnderBaseChange P` iff `(RingHom.toMorphismProperty P).IsStableUnderCobaseChange`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
49/0 Mathlib/Algebra/Category/Ring/Constructions.lean,Mathlib/RingTheory/IsTensorProduct.lean,Mathlib/RingTheory/RingHomProperties.lean 3 1 ['github-actions'] joelriou
assignee:joelriou
0-83957
23 hours ago
9-54333
9 days ago
9-54315
9 days
26693 euprunin
author:euprunin
chore: golf Computability/ using `grind` maintainer-merge t-computability 5/24 Mathlib/Computability/Language.lean,Mathlib/Computability/Partrec.lean,Mathlib/Computability/PostTuringMachine.lean,Mathlib/Computability/Primrec.lean,Mathlib/Computability/RegularExpressions.lean 5 8 ['euprunin', 'github-actions', 'grunweg', 'leanprover-bot', 'leanprover-community-mathlib4-bot'] YaelDillies
assignee:YaelDillies
0-82379
22 hours ago
0-82379
22 hours ago
29-12615
29 days
27024 grunweg
author:grunweg
feat: Gram-Schmidt orthonormalisation for sections of a vector bundle Add a parametrised version of Gram-Schmidt, for sections of a topological vector bundle with a bundle metric. This will be used to define orthonormal local frames. From the path towards geodesics and the Levi-Civita connection. Co-authored-by: Patrick Massot --- - [x] depends on: #27023 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-differential-geometry 279/11 Mathlib.lean,Mathlib/Analysis/InnerProductSpace/GramSchmidtOrtho.lean,Mathlib/Topology/VectorBundle/GramSchmidtOrtho.lean,scripts/noshake.json 4 67 ['faenuccio', 'github-actions', 'grunweg', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'sgouezel'] sgouezel
assignee:sgouezel
0-82369
22 hours ago
15-81448
15 days ago
16-2598
16 days
27711 wwylele
author:wwylele
feat(Algebra/Order): Add Add/Mul/Linear equiv versions of toLex/ofLex --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
84/30 Mathlib.lean,Mathlib/Algebra/Order/Group/Equiv.lean,Mathlib/Algebra/Order/GroupWithZero/Lex.lean,Mathlib/Algebra/Order/Module/Equiv.lean 4 7 ['github-actions', 'pechersky', 'wwylele'] nobody
0-78511
21 hours ago
1-67316
1 day ago
1-71896
1 day
27244 xroblot
author:xroblot
feat(RingTheory/DedekindDomain): lifting an ideal in an extension is injective This PR develops some API for [FractionalIdeal.extended](https://leanprover-community.github.io/mathlib4_docs/Mathlib/RingTheory/FractionalIdeal/Extended.html#FractionalIdeal.extended) and in particular for when it is an injective map (for an algebra map). As a consequence, it deduces the fact that lifting an integral ideal in an extension of Dedekind domains is an injective map. Note: the import increase happens in a leaf file `Mathlib.RingTheory.FractionalIdeal.Extended` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-algebra
label:t-algebra$
190/5 Mathlib/RingTheory/DedekindDomain/Ideal/Lemmas.lean,Mathlib/RingTheory/FractionalIdeal/Extended.lean,Mathlib/RingTheory/Localization/Basic.lean 3 2 ['github-actions', 'leanprover-community-bot-assistant'] nobody
0-77188
21 hours ago
0-77397
21 hours ago
14-40291
14 days
27792 kim-em
author:kim-em
feat: plumbing version of ClearExcept tactic t-meta 17/8 Mathlib/Tactic/ClearExcept.lean 1 1 ['github-actions'] nobody
0-77001
21 hours ago
0-77015
21 hours ago
0-77061
21 hours
27105 xroblot
author:xroblot
feat(Ring/DedekindDomain): formula for the splitting of prime ideals in an extension This PR just puts together all the results that were already there to deduce: ```lean map (algebraMap S R) p = ∏ P ∈ p.primesOver R, P ^ p.ramificationIdx (algebraMap S R) P ``` for `p` a maximal ideal of a ring `S` and `R` an extension of `S` that is a Dedekind ring. Note. There is a significant import increase in the file `RingTheory.DedekindDomain.Factorization`. However, this file is almost a leaf file so this increase only affects a limited number of files. If the increase is too big, a new file, say `RingTheory.DedekindDomain.PrimeSplitting`, can be added instead. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-algebra t-number-theory
label:t-algebra$
89/3 Mathlib/RingTheory/DedekindDomain/Factorization.lean,Mathlib/RingTheory/DedekindDomain/Ideal/Basic.lean,Mathlib/RingTheory/DedekindDomain/Ideal/Lemmas.lean,Mathlib/RingTheory/Ideal/Operations.lean,Mathlib/RingTheory/Ideal/Over.lean 5 2 ['github-actions', 'leanprover-community-bot-assistant'] nobody
0-75720
21 hours ago
0-75743
21 hours ago
18-46692
18 days
26101 xroblot
author:xroblot
feat(NumberField): specialized version of Kummer Dedekind for the splitting of prime numbers We prove a specialized version of [KummerDedekind.normalizedFactorsMapEquivNormalizedFactorsMinPolyMk](https://leanprover-community.github.io/mathlib4_docs/Mathlib/NumberTheory/KummerDedekind.html#KummerDedekind.normalizedFactorsMapEquivNormalizedFactorsMinPolyMk) for the splitting of rational prime numbers in number fields. This PR continues the work from #25038. --- - [ ] depends on: #26137 t-number-theory 173/2 Mathlib/NumberTheory/NumberField/Ideal/KummerDedekind.lean,Mathlib/NumberTheory/RamificationInertia/Basic.lean,Mathlib/RingTheory/AdjoinRoot.lean,Mathlib/RingTheory/DedekindDomain/Ideal/Lemmas.lean,Mathlib/RingTheory/Ideal/Over.lean 5 5 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'xroblot'] nobody
0-73715
20 hours ago
0-75388
20 hours ago
0-50
50 seconds
27055 wwylele
author:wwylele
feat(RingTheory): add HahnSeries.trunc --- This is for the proof of Hahn embedding theorem #27043, but it feels niche to have it in HahnSeries file, so I am not sure... if this doesn't feel right, I could make them private to the proof. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) maintainer-merge t-algebra
label:t-algebra$
53/0 Mathlib/RingTheory/HahnSeries/Addition.lean,Mathlib/RingTheory/HahnSeries/Basic.lean 2 6 ['Ruben-VandeVelde', 'ScottCarnahan', 'github-actions', 'kbuzzard', 'wwylele'] nobody
0-71488
19 hours ago
6-53419
6 days ago
19-67912
19 days
27794 xroblot
author:xroblot
feat(RingTheory): add `symm_apply_eq` and `eq_symm_apply` for `RingEquiv` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra easy
label:t-algebra$
6/0 Mathlib/Algebra/Ring/Equiv.lean 1 1 ['github-actions'] nobody
0-69967
19 hours ago
0-69980
19 hours ago
0-70024
19 hours
27442 artie2000
author:artie2000
feat(RingTheory/NonUnitalSubsemiring): add Aesop rules for `-(x * y)` subsemiring membership The Aesop rule `mul_mem` doesn't decompose goals of the form `-x * y ∈ s` or `x * -y ∈ s` in the absence of `neg_mem` because these expressions simplify to `-(x * y) ∈ s`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) maintainer-merge t-algebra
label:t-algebra$
22/1 Mathlib/RingTheory/NonUnitalSubsemiring/Defs.lean 1 20 ['Vierkantor', 'YaelDillies', 'artie2000', 'eric-wieser', 'github-actions'] YaelDillies
assignee:YaelDillies
0-20330
5 hours ago
3-13706
3 days ago
6-61674
6 days
27622 ShreckYe
author:ShreckYe
feat(Analysis/SpecialFunctions/Trigonometric): add the missing `tan_sub` and `tan_sub'` functions for both real and complex numbers While working on some proofs, I found that the `tan_sub` theorems are missing, while there are the corresponding`sin_sub` and `cos_sub` theorems. So I'd like to propose adding these for `tan`. new-contributor t-analysis 38/0 Mathlib/Analysis/SpecialFunctions/Trigonometric/Arctan.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Complex.lean 2 4 ['Ruben-VandeVelde', 'ShreckYe', 'github-actions', 'leanprover-community-bot-assistant'] nobody
0-65897
18 hours ago
0-65914
18 hours ago
3-15703
3 days
27790 pechersky
author:pechersky
feat(Topology): `IsDenseInducing.isUniformInducing_extend` extending along a uniform inducing function with another uniform inducing function with dense ranges of both creates a uniform inducing extension golfs a proof in #27696 and discussed in https://leanprover.zulipchat.com/#narrow/channel/217875-Is-there-code-for-X.3F/topic/isUniformInducing_extension --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology 62/0 Mathlib/Topology/DenseEmbedding.lean,Mathlib/Topology/UniformSpace/AbstractCompletion.lean,Mathlib/Topology/UniformSpace/Completion.lean,Mathlib/Topology/UniformSpace/UniformEmbedding.lean 4 2 ['github-actions', 'plp127'] nobody
0-63436
17 hours ago
0-84518
23 hours ago
0-84549
23 hours
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/) t-algebra t-topology t-number-theory
label:t-algebra$
106/20 Mathlib/RingTheory/Valuation/ValuativeRel.lean,Mathlib/Topology/Algebra/Valued/ValuativeRel.lean 2 2 ['github-actions', 'mathlib4-merge-conflict-bot'] nobody
0-60327
16 hours ago
0-62751
17 hours ago
17-14406
17 days
26885 pechersky
author:pechersky
feat(Topology/ValuativeRel): ValuativeTopology 𝒪[K] and even when not a field, `ValuativeRel 𝒪[K]` This is an example of something achievable with the new declarations that wasn't possible with Valued Such that we can discuss the valuations on the subring without always using coercions But to achieve this, one needs some juggling of the value groups --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) - [x] depends on: #26834 t-algebra t-topology t-number-theory
label:t-algebra$
74/1 Mathlib/RingTheory/Valuation/ValuativeRel.lean,Mathlib/Topology/Algebra/Valued/ValuativeRel.lean 2 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mathlib4-merge-conflict-bot'] alreadydone
assignee:alreadydone
0-59470
16 hours ago
0-62877
17 hours ago
24-19212
24 days
27492 euprunin
author:euprunin
chore: further golf some previously `grind` golfed proofs Replaces #27431, #27426, #27408 and #27404. It is probably safer to go with local `grind [t1, t2, …]` for now and leave global `@[grind =, etc.] theorem t1 …` annotations for later. I guess the local `grind [t1, t2, …]` uses can help guide which `t1`, `t2`, etc are worth to annotate "globally". 8/30 Mathlib/Algebra/BigOperators/Group/Finset/Basic.lean,Mathlib/LinearAlgebra/LinearPMap.lean,Mathlib/RingTheory/DividedPowers/Basic.lean,Mathlib/Topology/EMetricSpace/BoundedVariation.lean 4 6 ['github-actions', 'kim-em', 'leanprover-bot', 'mathlib-bors'] nobody
0-56402
15 hours ago
0-56423
15 hours ago
6-77215
6 days
27577 bjornsolheim
author:bjornsolheim
feat(Data/Fin/Tuple): lemmas on appending finite sequences Prove simple results regarding appending and de-appending of finite sequences. Used to define conical combinations and the conical hull (subsequent PR). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data new-contributor 42/0 Mathlib/Data/Fin/Tuple/Basic.lean 1 19 ['YaelDillies', 'bjornsolheim', 'eric-wieser', 'github-actions'] nobody
0-55943
15 hours ago
0-55943
15 hours ago
2-14927
2 days
27802 euprunin
author:euprunin
chore(Algebra): golf using the `have […] := by grind` pattern t-algebra
label:t-algebra$
4/9 Mathlib/Algebra/CharP/Defs.lean,Mathlib/Algebra/Lie/Engel.lean,Mathlib/Algebra/Order/BigOperators/Ring/Finset.lean 3 1 ['github-actions'] nobody
0-55255
15 hours ago
0-55264
15 hours ago
0-55312
15 hours
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/) 139/0 Archive.lean,Archive/Examples/Local/Laurent.lean,Archive/Examples/Local/NumberField.lean,Archive/Examples/Local/Padic.lean,Archive/Examples/Local/Witt.lean 5 1 ['github-actions'] nobody
0-54848
15 hours ago
19-25537
19 days ago
19-25519
19 days
27777 grunweg
author:grunweg
chore(Algebra/Group/Support): rename primed lemmas to match naming convention `mulSupport_inv` should be called `mulSupport_fun_inv`, according to the [naming convention](https://leanprover-community.github.io/contribute/naming.html#unexpanded-and-expanded-forms-of-functions), similarly for the other lemmas. Unfortunately, there is no good tooling yet for renames `A -> B` and `B -> C`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) maintainer-merge t-algebra
label:t-algebra$
42/28 Mathlib/Algebra/BigOperators/Finprod.lean,Mathlib/Algebra/Group/Indicator.lean,Mathlib/Algebra/Group/Support.lean,Mathlib/Algebra/GroupWithZero/Indicator.lean,Mathlib/LinearAlgebra/RootSystem/Base.lean,Mathlib/MeasureTheory/Function/SimpleFunc.lean,Mathlib/MeasureTheory/Function/StronglyMeasurable/Basic.lean,Mathlib/RingTheory/HahnSeries/Addition.lean,Mathlib/RingTheory/HahnSeries/Basic.lean,Mathlib/Topology/Algebra/Support.lean,Mathlib/Topology/LocallyFinsupp.lean 11 4 ['YaelDillies', 'github-actions', 'grunweg'] nobody
0-54652
15 hours ago
0-54652
15 hours ago
1-1794
1 day
26403 riccardobrasca
author:riccardobrasca
feat: add `isPrincipalIdealRing_of_isPrincipal_of_lt_or_isPrincipal_of_mem_primesOver_of_mem_Icc` This PR continues the work from #25186. Original PR: https://github.com/leanprover-community/mathlib4/pull/25186 t-number-theory 48/12 Mathlib/NumberTheory/NumberField/ClassNumber.lean 1 5 ['github-actions', 'grunweg', 'loefflerd', 'riccardobrasca', 'xroblot'] nobody
0-53097
14 hours ago
37-26606
1 month ago
37-26638
37 days
26142 YaelDillies
author:YaelDillies
chore(GeomSum): split into ring vs field and non-ordered vs ordered parts The motivation here is that `Data.Nat.Multiplicity` needs the results about geometric sums of naturals, without wanting to know anything about fields. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
705/634 Archive/Imo/Imo1982Q3.lean,Archive/Imo/Imo2013Q5.lean,Archive/Wiedijk100Theorems/PerfectNumbers.lean,Counterexamples/ZeroDivisorsInAddMonoidAlgebras.lean,Mathlib.lean,Mathlib/Algebra/Field/GeomSum.lean,Mathlib/Algebra/GeomSum.lean,Mathlib/Algebra/Order/CauSeq/BigOperators.lean,Mathlib/Algebra/Order/Field/GeomSum.lean,Mathlib/Algebra/Order/Ring/GeomSum.lean,Mathlib/Algebra/Ring/GeomSum.lean,Mathlib/Analysis/Polynomial/CauchyBound.lean,Mathlib/Analysis/SpecificLimits/Basic.lean,Mathlib/Analysis/SpecificLimits/FloorPow.lean,Mathlib/Combinatorics/Colex.lean,Mathlib/Combinatorics/SetFamily/KruskalKatona.lean,Mathlib/Data/Nat/Multiplicity.lean,Mathlib/LinearAlgebra/Projectivization/Cardinality.lean,Mathlib/LinearAlgebra/Vandermonde.lean,Mathlib/NumberTheory/Basic.lean,Mathlib/NumberTheory/FactorisationProperties.lean,Mathlib/NumberTheory/MulChar/Basic.lean,Mathlib/NumberTheory/Multiplicity.lean,Mathlib/RingTheory/AdicCompletion/Basic.lean,Mathlib/RingTheory/Ideal/Quotient/Index.lean,Mathlib/RingTheory/Idempotents.lean,Mathlib/RingTheory/IntegralDomain.lean,Mathlib/RingTheory/Nilpotent/Basic.lean,Mathlib/RingTheory/Polynomial/Basic.lean,Mathlib/Tactic/NormNum/Irrational.lean 30 3 ['github-actions', 'leanprover-community-bot-assistant'] joelriou
assignee:joelriou
0-52840
14 hours ago
1-54002
1 day ago
43-921
43 days
26989 joelriou
author:joelriou
feat(CategoryTheory): Artinian objects The API for Noetherian objects (from `Subobject.NoetherianObject`) is "dualized" in order to develop an API for Artinian objects. The previously existing definitions `ArtinianObject` and `NoetherianObject` from the file `CategoryTheory.Noetherian` are deprecated. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import maintainer-merge t-category-theory 178/64 Mathlib.lean,Mathlib/CategoryTheory/Noetherian.lean,Mathlib/CategoryTheory/Subobject/ArtinianObject.lean,Mathlib/CategoryTheory/Subobject/NoetherianObject.lean 4 13 ['github-actions', 'javra', 'joelriou', 'robin-carlier'] robin-carlier
assignee:robin-carlier
0-50352
13 hours ago
0-59049
16 hours ago
21-6428
21 days
25002 YaelDillies
author:YaelDillies
chore(Finsupp): move order properties under `Order` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import 360/326 Mathlib.lean,Mathlib/Algebra/Group/Finsupp.lean,Mathlib/Algebra/MvPolynomial/Basic.lean,Mathlib/Algebra/Order/Floor/Div.lean,Mathlib/Data/Finsupp/Ext.lean,Mathlib/Data/Finsupp/Multiset.lean,Mathlib/Data/Finsupp/Order.lean,Mathlib/Data/Finsupp/PWO.lean,Mathlib/Data/Finsupp/Pointwise.lean,Mathlib/Data/Finsupp/SMulWithZero.lean,Mathlib/Data/Finsupp/Single.lean,Mathlib/Data/Finsupp/Weight.lean,Mathlib/Data/List/ToFinsupp.lean,Mathlib/Data/Nat/Choose/Multinomial.lean,Mathlib/Data/Nat/Factorization/Defs.lean,Mathlib/Order/Preorder/Finsupp.lean 16 7 ['bryangingechen', 'github-actions', 'leanprover-community-bot-assistant'] bryangingechen
assignee:bryangingechen
0-49352
13 hours ago
6-44430
6 days ago
43-25706
43 days
26843 vasnesterov
author:vasnesterov
feat(Tactic/Simproc): nested quantifiers in `existsAndEq` Generalize the `existsAndEq` simproc to nested existential quantifiers. For example `∃ a, p a ∧ ∃ b, a = f b ∧ q b` now simplifies to `∃ b, p (f b) ∧ q b`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) This PR continues the work from #23365. Original PR: https://github.com/leanprover-community/mathlib4/pull/23365 migrated-from-branch large-import t-meta 452/73 Mathlib/Data/List/ProdSigma.lean,Mathlib/Tactic/Simproc/ExistsAndEq.lean,MathlibTest/Simproc/ExistsAndEq.lean 3 10 ['JovanGerb', 'github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'leanprover-community-mathlib4-bot', 'mathlib4-merge-conflict-bot', 'vasnesterov'] kmill
assignee:kmill
0-48837
13 hours ago
0-48860
13 hours ago
25-34599
25 days
27805 euprunin
author:euprunin
chore(Algebra/Order): golf `mem_piAntidiag` and `trichotomy_of_mul_eq_mul` using `grind` maintainer-merge t-algebra
label:t-algebra$
3/3 Mathlib/Algebra/Order/Antidiag/Pi.lean,Mathlib/Algebra/Order/Monoid/Unbundled/Basic.lean 2 2 ['github-actions', 'grunweg'] nobody
0-46109
12 hours ago
0-46109
12 hours ago
0-48212
13 hours
27803 euprunin
author:euprunin
chore(Algebra/ContinuedFractions): golf `fib_le_of_contsAux_b`, `sub_convs_eq` and `abs_sub_convs_le` using `grind` maintainer-merge t-algebra
label:t-algebra$
3/20 Mathlib/Algebra/ContinuedFractions/Computation/Approximations.lean 1 2 ['github-actions', 'grunweg'] nobody
0-46087
12 hours ago
0-46087
12 hours ago
0-48540
13 hours
27801 euprunin
author:euprunin
chore(Algebra/Order+Polynomial): golf entire `sub_self_div_two`, `div_two_sub_self`, `add_two_le_iff_lt_of_even_sub` and `natDegree_pos_of_nextCoeff_ne_zero` using `grind` maintainer-merge t-algebra
label:t-algebra$
4/9 Mathlib/Algebra/Order/Field/Basic.lean,Mathlib/Algebra/Order/Ring/Int.lean,Mathlib/Algebra/Polynomial/Degree/Lemmas.lean 3 2 ['github-actions', 'grunweg'] nobody
0-46064
12 hours ago
0-46064
12 hours ago
0-55749
15 hours
27640 Louddy
author:Louddy
feat(RatFunc): liftAlgebra and rank Add analogous results from `FractionRing` in the special case of `RatFunc`. This is needed as `RatFunc` is a one-field-struct. The first three are scoped instances lifting structure from `K[X]` to `RatFunc K`. Our application is two results stating that with appropriate context, the rank of `RatFunc K` over `RatFunc k` is the rank of `K` over `k`. - `RatFunc.liftAlgebra` ([`FractionRing`version](https://leanprover-community.github.io/mathlib4_docs/Mathlib/RingTheory/Localization/FractionRing.html#FractionRing.liftAlgebra)) - `RatFunc.isScalarTower_liftAlgebra` ([`FractionRing` version](https://leanprover-community.github.io/mathlib4_docs/Mathlib/RingTheory/Localization/FractionRing.html#FractionRing.isScalarTower_liftAlgebra)) - `RatFunc.faithfulSMul'` ([`FractionRing` version](https://leanprover-community.github.io/mathlib4_docs/Mathlib/RingTheory/Localization/FractionRing.html#FractionRing.instFaithfulSMul)) - `RatFunc.rank_ratFunc_ratFunc` (mathlib has a version for [`FractionRing`](https://leanprover-community.github.io/mathlib4_docs/Mathlib/RingTheory/Algebraic/Integral.html#Algebra.IsAlgebraic.rank_fractionRing_polynomial) but we use the version for [`IsFractionRing`](https://leanprover-community.github.io/mathlib4_docs/Mathlib/RingTheory/Algebraic/Integral.html#Algebra.IsAlgebraic.rank_of_isFractionRing) combined with `rank_polynomial_polynomial`.) - `RatFunc.finrank_ratFunc_ratFunc` The first three are declared as scoped instances of `RatFunc`. This creates a conflict with the current `LaurentSeries` file. To fix this, I have refactored to use the algebra instance coming from `RatFunc.liftAlgebra` instead of the `coeAlgHom` map defined in `LaurentSeries`. This has two main effects: - It simplifies the file. - The instance `RatFunc.instCoePolynomial` does not need to be hidden anymore. Looking forward to feedback! Xavier Co-authored-by: María Inés de Frutos Fernández <[mariaines.dff@gmail.com](mailto:mariaines.dff@gmail.com)> --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-algebra
label:t-algebra$
76/106 Mathlib/FieldTheory/RatFunc/Basic.lean,Mathlib/RingTheory/LaurentSeries.lean 2 1 ['github-actions'] nobody
0-44406
12 hours ago
0-44406
12 hours ago
0-47991
13 hours
27807 grunweg
author:grunweg
chore: mark Polynomial.differential fun_prop And remove a superfluous `local fun_prop` tag: Complex.continuous_abs is already marked fun_prop. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) easy 1/3 Mathlib/Analysis/Calculus/Deriv/Polynomial.lean,Mathlib/NumberTheory/Transcendental/Lindemann/AnalyticalPart.lean 2 1 ['github-actions'] nobody
0-42963
11 hours ago
0-43030
11 hours ago
0-43014
11 hours
27809 euprunin
author:euprunin
chore(Algebra/Module): golf `eq_zero_of_ofSpanSingleton_apply_self` using `grind […]` t-algebra
label:t-algebra$
4/12 Mathlib/Algebra/Module/CharacterModule.lean 1 1 ['github-actions'] nobody
0-41869
11 hours ago
0-42324
11 hours ago
0-42369
11 hours
27804 euprunin
author:euprunin
chore(Algebra/Polynomial): golf `coeff_mul_natTrailingDegree_add_natTrailingDegree` and `div_eq_quo_add_sum_rem_div` using `grind [Finset.*]` maintainer-merge t-algebra
label:t-algebra$
3/13 Mathlib/Algebra/Polynomial/Degree/TrailingDegree.lean,Mathlib/Algebra/Polynomial/PartialFractions.lean 2 2 ['github-actions', 'grunweg'] nobody
0-41829
11 hours ago
0-46097
12 hours ago
0-48373
13 hours
27781 euprunin
author:euprunin
chore(Topology/Algebra): golf `prod_subset` using `grind [Set.*]` t-topology 2/4 Mathlib/Topology/Algebra/Nonarchimedean/Basic.lean 1 1 ['github-actions'] nobody
0-41727
11 hours ago
1-7120
1 day ago
1-7171
1 day
27628 EtienneC30
author:EtienneC30
feat(ProbabilityTheory): a new predicate HasLaw Introduce a predicate `HasLaw X μ P` stating that the random variable `X` has law `μ` under the measure `P`. This is expressed as `P.map X = μ`. We also require `X` to be `P`-almost-everywhere measurable to avoid pathological cases. from BrownianMotion --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-measure-probability 128/0 Mathlib.lean,Mathlib/Probability/HasLaw.lean 2 6 ['DavidLedvinka', 'EtienneC30', 'github-actions', 'kex-y'] nobody
0-41660
11 hours ago
3-45137
3 days ago
3-45120
3 days
27728 euprunin
author:euprunin
chore(Data/Complex): golf `norm_exp_sub_sum_le_norm_mul_exp` using `grind [Finset.*]` t-data maintainer-merge 1/4 Mathlib/Data/Complex/Exponential.lean 1 2 ['github-actions', 'grunweg'] nobody
0-41619
11 hours ago
1-36319
1 day ago
1-48165
1 day
27563 euprunin
author:euprunin
chore(Topology/EMetricSpace/BoundedVariation): golf `add_le_union` using `grind [Finset.*]` t-topology 2/13 Mathlib/Topology/EMetricSpace/BoundedVariation.lean 1 1 ['github-actions'] nobody
0-41576
11 hours ago
5-7788
5 days ago
5-7837
5 days
27561 euprunin
author:euprunin
chore(Topology/EMetricSpace/BoundedVariation): golf `add_point` using `grind [Finset.*]` t-topology 5/26 Mathlib/Topology/EMetricSpace/BoundedVariation.lean 1 1 ['github-actions'] nobody
0-41554
11 hours ago
5-9154
5 days ago
5-9203
5 days
24889 Kha
author:Kha
chore: do not include cache requests in build benchmark 5/2 scripts/bench/temci-config.run.yml 1 4 ['Kha', 'github-actions', 'leanprover-bot'] MichaelStollBayreuth
assignee:MichaelStollBayreuth
0-40695
11 hours ago
79-44689
2 months ago
79-44669
79 days
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/) t-algebraic-geometry 251/0 Mathlib.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Affine/Basic.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Singular/Node.lean 3 11 ['Multramate', 'acmepjz', 'erdOne', 'github-actions'] kim-em
assignee:kim-em
0-40690
11 hours ago
72-69364
2 months ago
72-69418
72 days
25861 robin-carlier
author:robin-carlier
feat(CategoryTheory/Monoidal/Action): action of opposite categories Given a monoidal category `C` and a category `D`, we show that left (resp. right) `C`-actions on `D` induce left (resp. right) `Cᵒᵖ`-actions on `Dᵒᵖ`. Conversely, we show that left/right actions of `Cᵒᵖ` on `Dᵒᵖ` induce left/right actions of `C` on `D`. --- - [ ] depends on: #25860 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory 272/0 Mathlib/CategoryTheory/Monoidal/Action/Opposites.lean 1 4 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] joelriou
assignee:joelriou
0-40686
11 hours ago
27-26954
27 days ago
27-31230
27 days
25907 mans0954
author:mans0954
Low order roots of unity This PR continues the work from #25470. Original PR: https://github.com/leanprover-community/mathlib4/pull/25470 t-algebra
label:t-algebra$
182/0 Mathlib/Algebra/CharP/Invertible.lean,Mathlib/RingTheory/RootsOfUnity/Complex.lean 2 2 ['github-actions', 'mans0954'] kim-em
assignee:kim-em
0-40683
11 hours ago
47-33371
1 month ago
47-33420
47 days
26000 Hagb
author:Hagb
feat(RingTheory/MvPolynomial/MonomialOrder): some lemmas about degree Co-authored-by: Hao Shen @tsuki8 <3118181069@qq.com> --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
24/0 Mathlib/RingTheory/MvPolynomial/MonomialOrder.lean 1 6 ['Hagb', 'Ruben-VandeVelde', 'github-actions'] riccardobrasca
assignee:riccardobrasca
0-40680
11 hours ago
28-27871
28 days ago
42-34051
42 days
26054 FMLJohn
author:FMLJohn
feat(RingTheory/GradedAlgebra/Homogeneous/Subsemiring): homogeneous subsemirings of a graded semiring --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) In this pull request, we have defined homogeneous subsemirings of `GradedRing 𝒜` where `𝒜 : ι → σ`, `SetLike σ A` and `AddSubmonoidClass σ A`. ## Main definitions For any `R : Subsemiring A`: * `Subsemiring.IsHomogeneous 𝒜 R`: The property that a subsemiring is closed under `GradedRing.proj`. * `HomogeneousSubsemiring 𝒜`: The structure extending subsemirings which satisfy `Subsemiring.IsHomogeneous`. t-algebra
label:t-algebra$
120/0 Mathlib.lean,Mathlib/RingTheory/GradedAlgebra/Homogeneous/Subsemiring.lean 2 1 ['github-actions'] kim-em
assignee:kim-em
0-40675
11 hours ago
45-11979
1 month ago
45-11962
45 days
26351 RemyDegenne
author:RemyDegenne
feat: covering and packing numbers of sets in a metric space We define covering numbers of sets in a pseudo-metric space, which are minimal cardinalities of `ε`-covers of sets. We also define the packing number, which is the maximal cardinality of an `ε`-separated set. From the Brownian motion project. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology 261/0 Mathlib.lean,Mathlib/Topology/MetricSpace/CoveringNumbers.lean 2 4 ['ADedecker', 'YaelDillies', 'github-actions'] j-loreaux
assignee:j-loreaux
0-40670
11 hours ago
38-43203
1 month ago
38-43248
38 days
26396 xroblot
author:xroblot
feat(RingTheory): define the dual of a basis for the trace and prove basic properties --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
120/37 Mathlib/LinearAlgebra/BilinearForm/Properties.lean,Mathlib/RingTheory/DedekindDomain/Different.lean,Mathlib/RingTheory/Trace/Basic.lean 3 1 ['github-actions'] adomani
assignee:adomani
0-40668
11 hours ago
37-48675
1 month ago
37-48724
37 days
26655 Rida-Hamadani
author:Rida-Hamadani
feat(SimpleGraph): sub-walks defines (contiguous) subwalks and provides lemmas about them. Co-authored-by: Kyle Miller Co-authored-by: Vlad Tsyrklevich --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics 176/0 Mathlib/Combinatorics/SimpleGraph/Paths.lean,Mathlib/Combinatorics/SimpleGraph/Walk.lean,Mathlib/Data/List/Infix.lean 3 20 ['Rida-Hamadani', 'github-actions', 'jt496', 'kmill', 'vlad902'] awainverse
assignee:awainverse
0-40667
11 hours ago
29-49241
29 days ago
29-49291
29 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 t-algebra t-analysis t-number-theory
label:t-algebra$
238/25 Mathlib.lean,Mathlib/Analysis/Normed/ValuativeRel.lean,Mathlib/Topology/Algebra/Valued/ValuativeRel.lean 3 11 ['ADedecker', 'adamtopaz', 'github-actions', 'mathlib4-dependent-issues-bot', 'pechersky'] kbuzzard
assignee:kbuzzard
0-40663
11 hours ago
25-10044
25 days ago
25-10307
25 days
26875 michaellee94
author:michaellee94
feat(Manifold/PartitionOfUnity): existence of global C^n smooth section for nontrivial bundles Add existence of global C^n smooth section for nontrivial bundles --- - [x] depends on: #26671 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-differential-geometry 121/14 Mathlib/Geometry/Manifold/PartitionOfUnity.lean 1 8 ['github-actions', 'grunweg', 'mathlib4-dependent-issues-bot', 'michaellee94'] ocfnash
assignee:ocfnash
0-40661
11 hours ago
22-15460
22 days ago
22-30131
22 days
27047 YaelDillies
author:YaelDillies
feat: `MonoidHom.toAdditive''` as a `MulEquiv` From Toric --- I haven't yet been very thorough with the new lemmas. I first want to hear thoughts about the names [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) toric t-algebra
label:t-algebra$
31/7 Mathlib/Algebra/Group/TypeTags/Hom.lean 1 1 ['github-actions'] adomani
assignee:adomani
0-40658
11 hours ago
19-54538
19 days ago
19-86395
19 days
27308 xyzw12345
author:xyzw12345
feat(LinearAlgebra/SymmetricAlgebra): IsSymmetricAlgebra This PR continues the work from #24602. Original PR: https://github.com/leanprover-community/mathlib4/pull/24602 t-algebra
label:t-algebra$
78/0 Mathlib/LinearAlgebra/SymmetricAlgebra/Basic.lean,Mathlib/LinearAlgebra/SymmetricAlgebra/Basis.lean 2 1 ['github-actions'] mattrobball
assignee:mattrobball
0-40656
11 hours ago
12-25254
12 days ago
12-25306
12 days
27439 Vierkantor
author:Vierkantor
chore(*): review 2024-04-01 adaptation notes There are three kinds of adaptation notes from the changes on 2024-04-01. One about `erw` "blowing up"; this referred to a backwards compatibility flag that was already removed long ago (#14064). So this can just be deleted. A few about needing to use `symm` before `ext` fires: this is because `apply` failing to unify when mixing very general limit definitions and very specific operations for equalizers/pullbacks. I propose we fix this by unfolding the terms manually in an `intro` type ascription. In the longer term we should consider instead specializing the limit lemmas to these specific shapes. A few about `aesop` not working. This has the same underlying cause, due to `ext` not applying, so it now looks like `intro s (m : _ --> _) x; aesop`. Same specializing of the limit lemmas may be useful here. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) tech debt 8/25 Mathlib/AlgebraicGeometry/Spec.lean,Mathlib/CategoryTheory/Limits/Shapes/KernelPair.lean,Mathlib/CategoryTheory/Limits/Shapes/Kernels.lean,Mathlib/CategoryTheory/Limits/Shapes/Products.lean 4 2 ['github-actions', 'grunweg'] jcommelin
assignee:jcommelin
0-40451
11 hours ago
8-13083
8 days ago
8-13066
8 days
26210 Thmoas-Guan
author:Thmoas-Guan
feat(RingTheory): associated primes of localized module We prove that `Ass(S^{-1}M)` is equal to the preimage of `Ass(M)` under `Ideal.comap` if the base ring is Noetherian. From this we conclude that every minimal prime over `Module.annihilator R M` is in `Ass(M)` when `M` is finitely generated. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-algebra
label:t-algebra$
79/17 Mathlib/RingTheory/Ideal/AssociatedPrime/Localization.lean 1 17 ['Thmoas-Guan', 'chrisflav', 'github-actions', 'mbkybky'] nobody
0-38275
10 hours ago
0-38526
10 hours ago
27-70547
27 days
26765 KiringYJ
author:KiringYJ
feat(MeasureTheory/PiSystem): add π-λ theorem and SetLike instance Add two small features to `MeasureTheory/PiSystem`: 1. SetLike instance `instance : SetLike (DynkinSystem α) (Set α)` This lets us write `s ⊆ d` and `t ∈ d` for a DynkinSystem `d`, matching usual mathlib style. 2. `DynkinSystem.pi_lambda` lemma Classical π‑λ theorem: if a π‑system `s` is contained in a Dynkin system `d`, every set measurable for `σ(s)` is also in `d`. Currently, mathlib exposes this result only indirectly (e.g. via `generateFrom_eq`). Although logically equivalent, it is not obvious at first glance that those lemmas are the π‑λ theorem. The new lemma states the result in its familiar textbook form, so users can recognise and cite it immediately. Both pieces are under 10 lines, term‑mode only, and do not modify existing APIs. No breaking changes. No dependencies. new-contributor t-measure-probability 13/0 Mathlib/MeasureTheory/PiSystem.lean 1 13 ['EtienneC30', 'KiringYJ', 'github-actions', 'ocfnash'] nobody
0-38111
10 hours ago
1-23958
1 day ago
28-11801
28 days
27814 xroblot
author:xroblot
feat(FieldTheory/Galois): add `IsGalois.of_equiv_equiv` Assume that `E/F` is Galois and that `F ≃+* M` and `E ≃+* N` with some compatibility hypothesis, then `N/M` is Galois --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
32/0 Mathlib/Algebra/Polynomial/Eval/Degree.lean,Mathlib/FieldTheory/Galois/Basic.lean,Mathlib/FieldTheory/Minpoly/Field.lean,Mathlib/FieldTheory/Normal/Defs.lean 4 1 ['github-actions'] nobody
0-35782
9 hours ago
0-35788
9 hours ago
0-35834
9 hours
27816 BGuillemet
author:BGuillemet
feat(CategoryTheory/Sites/SheafOfTypes): composition of a sheaf with uliftFunctor is still a sheaf Prove that if a presheaf of types is a sheaf, then its composition with `uliftFunctor` is still a sheaf. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-category-theory 4/0 Mathlib/CategoryTheory/Sites/SheafOfTypes.lean 1 1 ['github-actions'] nobody
0-33454
9 hours ago
0-33490
9 hours ago
0-33512
9 hours
26914 quangvdao
author:quangvdao
feat(Data/PFunctor/Univariate): more definitions for univariate `PFunctor` This PR defines several basic definitions of `PFunctor`, including zero, one, constants, monomials, coproduct (sum), product, sigma, pi, tensor product, universe lifting, and equivalence. We also add: (1) simple lemmas connecting the basic definitions, (2) an automatically derived ext lemma for `PFunctor` via `@[ext]` attribute Some things I'm not clear on: - I define `HAdd` and `HMul` instances for coproduct and product of poly functors having different universe levels. Should I also define `Add` and `Mul` instances for poly functors having the same universe level? - Is it ok to define notation for tensor product, i.e. `@[inherit_doc] scoped infixr:80 " ⊗ " => tensor`? I'm worried it might clash with other notation. - Need a double-check on the priority of notation. Some future definitions to add: - Various equivalences arising from arithmetic identities, e.g., `P + 0 ≃ₚ P`. - Definitions of Lenses and Charts (each of them will be a file or even a folder) - Exponential objects (corresponding to both `prod` and `tensor`) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data 183/5 Mathlib/Data/PFunctor/Univariate/Basic.lean 1 12 ['alexkeizer', 'eric-wieser', 'github-actions', 'quangvdao'] nobody
0-33241
9 hours ago
23-75388
23 days ago
23-75433
23 days
27819 BGuillemet
author:BGuillemet
feat(CategoryTheory/Yoneda): add curried version of Yoneda lemma for heterogeneous universes, and other version of homNatIso Prove a curried version of `yonedaCompUliftFunctorEquiv`, ie a completely functorial version of the Yoneda lemma with heterogeneous universes. Dually, prove a curried version of `coyonedaCompUliftFunctorEquiv`, ie a completely functorial version of the coYoneda lemma with heterogeneous universes. In addition, prove a functorial version of `FullyFaithful.natEquiv` using `coyoneda` instead of `yoneda` (previously, the only functorial version of `FullyFaithful.natEquiv` were `homNatIso`, which is written using `yoneda`). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-category-theory 162/36 Mathlib/CategoryTheory/Yoneda.lean 1 1 ['github-actions'] nobody
0-32324
8 hours ago
0-32402
8 hours ago
0-32402
9 hours
27815 BGuillemet
author:BGuillemet
feat(CategoryTheory/Limits/Shapes/Products): add limMapPi and sigmaMapColim Add the canonical morphism from a limit to the product over its objects. Prove that it is a monomorphism. Dually, add the canonical morphism to a colimit from the coproduc of its objects and prove that it is an epimorphism. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-category-theory 44/0 Mathlib/CategoryTheory/Limits/Shapes/Products.lean 1 1 ['github-actions'] nobody
0-32090
8 hours ago
0-34018
9 hours ago
0-34043
9 hours
27820 FLDutchmann
author:FLDutchmann
chore(NumberTheory/SelbergSieve): turn `BoundingSieve` into a struct Based on a discussion [on zulip](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/BoundingSieve.20is.20a.20class.3F.3F). I wound up removing the custom notation as well, since not everybody was fond of it and I had some trouble getting it to work properly with structure inheritance and the corresponding coersions. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis t-number-theory 51/84 Mathlib/NumberTheory/SelbergSieve.lean 1 1 ['github-actions'] nobody
0-31137
8 hours ago
0-31160
8 hours ago
0-31195
8 hours
27823 Louddy
author:Louddy
feat(RatFunc): transcendental_X The variable `RatFunc.X` is transcendental of `K` in `RatFunc K`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
10/0 Mathlib/FieldTheory/RatFunc/AsPolynomial.lean 1 1 ['github-actions'] nobody
0-30305
8 hours ago
0-30315
8 hours ago
0-30360
8 hours
27822 Louddy
author:Louddy
feat(RatFunc): theorems algebraMap polynomial Two simple lemmas about the `algebraMap` from `F[X]` to `RatFunc F`: - A `monomial n a` is `C a * X ^ n` (here we are using `RatFunc.X` and `RatFunc.C`.) - The algebraMap from `F[X]` to `RatFunc F` is the same as the evaluation of a polynomial `p` at `RatFunc.X`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra easy
label:t-algebra$
9/0 Mathlib/FieldTheory/RatFunc/AsPolynomial.lean 1 1 ['github-actions'] nobody
0-30293
8 hours ago
0-30293
8 hours ago
0-30443
8 hours
27824 ChrisHughes24
author:ChrisHughes24
feat(Calculus): exists_gt_of_deriv_pos and variants --- I created a new file for this as I anticipate there will be many lemmas relating derivatives and monotonicity in future. Some lemmas relating deriviatives to monotonicity are already in mathlib and should maybe moved to the file (e.g. docs#HasDerivWithinAt.nonneg_of_monotoneOn). I stated them in as much generality as I could, copying the generality of `HasDerivWithinAt.nonneg_of_monotoneOn`. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis 94/0 Mathlib.lean,Mathlib/Analysis/Calculus/Deriv/Order.lean 2 1 ['github-actions'] nobody
0-30195
8 hours ago
0-30206
8 hours ago
0-30252
8 hours
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/) t-logic 618/0 Mathlib.lean,Mathlib/ModelTheory/FunctionalFormula.lean 2 3 ['ChrisHughes24', 'github-actions', 'mathlib4-dependent-issues-bot'] nobody
0-28771
7 hours ago
37-45187
1 month ago
37-45445
37 days
27284 FernandoChu
author:FernandoChu
Chore(CategoryTheory/MorphismProperty/MonoFactorization): Factor out mono factorizations Factored out `MonoFactorisations` from the `Images` file; also rename it to `MonoFactori*z*ations` so it's inline with the rest of Mathlib. I'm also sneaking in some very basic extremal epis results if you don't mind, these were meant to be used to prove ```lean instance (priority := 100) hasStrongEpiImages_of_hasPullbacks_of_hasEqualizers [HasPullbacks C] [HasEqualizers C] : HasStrongEpiImages C ``` Which I noticed too late already had a proof; I think the proof has been improved anyways, it's just `infer_instance` now. new-contributor t-category-theory 468/312 Mathlib.lean,Mathlib/Algebra/Category/Grp/Images.lean,Mathlib/Algebra/Category/ModuleCat/Images.lean,Mathlib/AlgebraicTopology/SimplexCategory/Basic.lean,Mathlib/CategoryTheory/Abelian/Basic.lean,Mathlib/CategoryTheory/Category/Factorisation.lean,Mathlib/CategoryTheory/ConcreteCategory/EpiMono.lean,Mathlib/CategoryTheory/Limits/Preserves/Shapes/Images.lean,Mathlib/CategoryTheory/Limits/Shapes/ExtremalEpi.lean,Mathlib/CategoryTheory/Limits/Shapes/Images.lean,Mathlib/CategoryTheory/Limits/Shapes/Kernels.lean,Mathlib/CategoryTheory/Limits/Shapes/StrongEpi.lean,Mathlib/CategoryTheory/Limits/Shapes/ZeroMorphisms.lean,Mathlib/CategoryTheory/Limits/Types/Images.lean,Mathlib/CategoryTheory/MorphismProperty/MonoFactorization.lean,Mathlib/CategoryTheory/Sites/Subsheaf.lean,Mathlib/Order/Category/NonemptyFinLinOrd.lean,scripts/nolints_prime_decls.txt 18 29 ['FernandoChu', 'github-actions', 'joelriou', 'robin-carlier'] TwoFX
assignee:TwoFX
0-28302
7 hours ago
0-28392
7 hours ago
13-31623
13 days
27825 yonggyuchoimath
author:yonggyuchoimath
feat(RingTheory/Ideal/Height): sup of ideal heights equals Krull dimension feat: sup of ideal heights equals Krull dimension --- This PR adds `Ideal.sup_height_eq_ringKrullDim` `Ideal.sup_primeHeight_eq_ringKrullDim` They show the suprema of heights of ideals / prime ideals are equal to the Krull dimension, when the ring is nonzero. new-contributor t-algebra
label:t-algebra$
53/0 Mathlib/RingTheory/Ideal/Height.lean 1 2 ['github-actions', 'yonggyuchoimath'] nobody
0-27921
7 hours ago
0-29520
8 hours ago
0-29568
8 hours
27785 staroperator
author:staroperator
chore(Algebra/Group/Submonoid): golf `Nat.addSubmonoid_closure_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/) bench-after-CI large-import t-algebra
label:t-algebra$
5/13 Mathlib/Algebra/Group/Submonoid/Membership.lean,Mathlib/Algebra/Group/Submonoid/Operations.lean,Mathlib/Algebra/Order/Star/Basic.lean 3 2 ['github-actions', 'staroperator'] nobody
0-27712
7 hours ago
1-6767
1 day ago
1-6872
1 day
27755 bwangpj
author:bwangpj
feat(RepresentationTheory/Basic): direct sum of representations Define the `DirectSum` of a family of `Representation`s. [Zulip thread](https://leanprover.zulipchat.com/#narrow/channel/116395-maths/topic/Representation.20Theory) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra
label:t-algebra$
39/0 Mathlib/RepresentationTheory/Basic.lean 1 3 ['bwangpj', 'github-actions', 'kbuzzard'] nobody
0-27390
7 hours ago
1-22233
1 day ago
1-22279
1 day
27828 Louddy
author:Louddy
feat(Algebra/Adjoin): singleton as aeval For `x : A`, elements of `Algebra.adjoin R {x}` can be represented as a polynomial of `R` evaluated at the point `x`. This PR introduces three (3) theorems related to this: - `adjoin_mem_exists_aeval` rewrite an element of `A` in `adjoin R {x}` as the `aeval` of some polynomial. - `adjoin_eq_exists_aeval` rewrite an element `adjoin R {x}` as the `aeval` of some polynomial. - `adjoin_singleton_induction`: an induction principle reducing problems over `adjoin R {x}` to problems of the form `M (⟨aeval x p, aeval_mem_adjoin_singleton R x⟩ : adjoin R {x})`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
29/8 Mathlib/RingTheory/Adjoin/Polynomial.lean 1 1 ['github-actions'] nobody
0-27150
7 hours ago
0-27152
7 hours ago
0-27204
7 hours
27749 EtienneC30
author:EtienneC30
feat: the covariance of independent random variables is 0 and consequences Simplify the proofs in `Probability/Integration` and move the file in the `Independence` folder (which is the main reason for the huge diff). Use this to prove that the covariance of independent random variables is 0. Use this to golf the proof that the variance of a sum of independent random variables is the sum of their variances. Also prove that random variables on a product space are independent. --- - [x] depends on: #27721 - [x] depends on: #27736 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-measure-probability 481/402 Mathlib.lean,Mathlib/MeasureTheory/Function/LpSeminorm/Basic.lean,Mathlib/MeasureTheory/Measure/Prod.lean,Mathlib/Probability/Independence/Basic.lean,Mathlib/Probability/Independence/Integration.lean,Mathlib/Probability/Integration.lean,Mathlib/Probability/Moments/Basic.lean,Mathlib/Probability/Moments/Covariance.lean,Mathlib/Probability/Moments/Variance.lean 9 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
0-25256
7 hours ago
0-25258
7 hours ago
0-26152
7 hours
27674 EtienneC30
author:EtienneC30
feat: integrability in a product space Prove that `f : (i : ι) → X → E i` is in `Lᵖ` if and only if for all `i`, `f i` is in `Lᵖ`. Do the same for `f : X → (E × F)`. Also provide `WithLp` versions. from BrownianMotion --- - [x] depends on: #27721 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-measure-probability 276/1 Mathlib.lean,Mathlib/Analysis/NormedSpace/OperatorNorm/NormedSpace.lean,Mathlib/MeasureTheory/Integral/Eval/Basic.lean,Mathlib/MeasureTheory/Integral/Eval/WithLp.lean,Mathlib/Topology/MetricSpace/Injection.lean 5 3 ['RemyDegenne', 'github-actions', 'mathlib4-dependent-issues-bot'] nobody
0-24586
6 hours ago
0-24586
6 hours ago
2-3837
2 days
26967 joelriou
author:joelriou
feat(AlgebraicTopology/ModelCategory): left homotopies This PR studies the notion of "left homotopy" given by cylinder objects in model categories. --- - [x] depends on: #26171 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebraic-topology t-category-theory 303/0 Mathlib.lean,Mathlib/AlgebraicTopology/ModelCategory/LeftHomotopy.lean 2 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] robin-carlier
assignee:robin-carlier
0-23782
6 hours ago
1-35002
1 day ago
10-17874
10 days
26958 joelriou
author:joelriou
feat(AlgebraicTopology): path objects in model categories This PR dualizes #26171 which was about cylinder objects. --- - [x] depends on: #26171 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebraic-topology t-category-theory 335/0 Mathlib.lean,Mathlib/AlgebraicTopology/ModelCategory/IsCofibrant.lean,Mathlib/AlgebraicTopology/ModelCategory/PathObject.lean,Mathlib/CategoryTheory/Limits/Shapes/Pullback/CommSq.lean 4 4 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] robin-carlier
assignee:robin-carlier
0-23747
6 hours ago
1-35007
1 day ago
10-51958
10 days
25829 kbuzzard
author:kbuzzard
feat: add mulEquivHaarChar API for the positive real factor by which an continuous multiplicative equivalence scales a regular Haar measure on a locally compact topological group. From FLT. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-measure-probability 158/0 Mathlib.lean,Mathlib/MeasureTheory/Group/Measure.lean,Mathlib/MeasureTheory/Measure/Haar/MulEquivHaarChar.lean,Mathlib/MeasureTheory/Measure/Haar/Unique.lean 4 18 ['RemyDegenne', 'github-actions', 'kbuzzard'] nobody
0-23402
6 hours ago
0-23474
6 hours ago
45-53412
45 days
26738 javra
author:javra
feat(AlgebraicToplogy/SimplexCategory): add notation for faces and degeneracies general truncated simplex categories --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebraic-topology infinity-cosmos 43/32 Mathlib/AlgebraicTopology/SimplexCategory/Truncated.lean,Mathlib/AlgebraicTopology/SimplicialSet/HomotopyCat.lean 2 4 ['emilyriehl', 'github-actions', 'leanprover-community-bot-assistant'] nobody
0-23148
6 hours ago
0-34233
9 hours ago
14-25235
14 days
27707 FLDutchmann
author:FLDutchmann
feat(NumberTheory/SelbergSieve): define Selberg's weights and prove basic results. This PR continues the work from #23635. Original PR: https://github.com/leanprover-community/mathlib4/pull/23635 t-analysis t-number-theory 407/83 Mathlib/NumberTheory/Divisors.lean,Mathlib/NumberTheory/SelbergSieve.lean 2 1 ['github-actions'] nobody
0-19145
5 hours ago
0-20169
5 hours ago
1-77075
1 day
27637 Louddy
author:Louddy
feat(Subalgebra): simp lemma for algebraMap mk Add three lemma (two simp) for the interaction of `Subalgebra.mk` and `algebraMap`. Let me know if you think these lemmas should be placed elsewhere. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
20/8 Mathlib/Algebra/Algebra/Subalgebra/Basic.lean,Mathlib/LinearAlgebra/CliffordAlgebra/Even.lean 2 14 ['Louddy', 'eric-wieser', 'github-actions'] nobody
0-19011
5 hours ago
3-21688
3 days ago
3-21680
3 days
27837 CBirkbeck
author:CBirkbeck
feat(NumberTheory/Divisors): add divisorAntidiagonal equivalence. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-number-theory 33/0 Mathlib/NumberTheory/Divisors.lean 1 1 ['github-actions'] nobody
0-18764
5 hours ago
0-18769
5 hours ago
0-18815
5 hours
27004 kbuzzard
author:kbuzzard
chore: rename doset to doubleCoset --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) I was working with these in FLT and something snapped. It's *not a word*. t-algebra
label:t-algebra$
105/41 Mathlib/GroupTheory/DoubleCoset.lean 1 9 ['eric-wieser', 'github-actions', 'grunweg', 'j-loreaux', 'kbuzzard'] nobody
0-18686
5 hours ago
0-18686
5 hours ago
0-43859
12 hours
27316 mans0954
author:mans0954
feature(Analysis/LocallyConvex/WeakDual): functional_mem_span_iff Sufficient and necessary conditions for a linear functional to be in the span of a finite set of linear functionals. This result is Rudin, Functional Analysis, Second edition, Lemma 3.9 (see also Bourbaki TVS, II.6 Proposition 5). A key application of this result is the proof that `WeakBilin.eval B` is surjective i.e. the dual of `E` with the weak topology is identified with `F`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-analysis 106/0 Mathlib/Analysis/LocallyConvex/WeakDual.lean,docs/references.bib 2 9 ['ADedecker', 'github-actions', 'mans0954'] nobody
0-18381
5 hours ago
4-8126
4 days ago
8-52354
8 days
27791 alreadydone
author:alreadydone
chore(Algebra/Regular): split Defs out of Basic and redefine IsCancelMul Redefine Is(Left/Right)CancelMul(Zero) in terms of Is(Left/Right)Regular. Defeq to the original defs except for argument explicitness/order. Part of #22997 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-algebra
label:t-algebra$
198/165 Archive/Imo/Imo2015Q6.lean,Mathlib.lean,Mathlib/Algebra/Group/Defs.lean,Mathlib/Algebra/Group/Prod.lean,Mathlib/Algebra/Group/TypeTags/Basic.lean,Mathlib/Algebra/Group/UniqueProds/Basic.lean,Mathlib/Algebra/GroupWithZero/Associated.lean,Mathlib/Algebra/GroupWithZero/Basic.lean,Mathlib/Algebra/GroupWithZero/Defs.lean,Mathlib/Algebra/GroupWithZero/InjSurj.lean,Mathlib/Algebra/GroupWithZero/Nat.lean,Mathlib/Algebra/GroupWithZero/Opposite.lean,Mathlib/Algebra/GroupWithZero/Regular.lean,Mathlib/Algebra/MonoidAlgebra/NoZeroDivisors.lean,Mathlib/Algebra/Order/Group/Basic.lean,Mathlib/Algebra/Order/Group/Bounds.lean,Mathlib/Algebra/Order/Group/Int/Sum.lean,Mathlib/Algebra/Order/Interval/Set/Instances.lean,Mathlib/Algebra/Order/Monoid/Unbundled/Basic.lean,Mathlib/Algebra/Order/Ring/Defs.lean,Mathlib/Algebra/Polynomial/Coeff.lean,Mathlib/Algebra/Regular/Basic.lean,Mathlib/Algebra/Regular/Defs.lean,Mathlib/Algebra/Regular/Opposite.lean,Mathlib/Algebra/Regular/Pi.lean,Mathlib/Algebra/Regular/Prod.lean,Mathlib/Algebra/Regular/SMul.lean,Mathlib/Algebra/Regular/ULift.lean,Mathlib/Algebra/Ring/Basic.lean,Mathlib/Algebra/Ring/Int/Defs.lean,Mathlib/Algebra/Ring/Regular.lean,Mathlib/Algebra/Star/Basic.lean,Mathlib/Data/Int/Interval.lean,Mathlib/Data/Int/Range.lean,Mathlib/Data/PNat/Basic.lean,Mathlib/GroupTheory/MonoidLocalization/MonoidWithZero.lean,Mathlib/Order/Interval/Finset/Box.lean,Mathlib/RingTheory/DedekindDomain/Ideal/Basic.lean,Mathlib/RingTheory/Localization/Defs.lean,Mathlib/SetTheory/Game/Impartial.lean,Mathlib/SetTheory/Nimber/Basic.lean,Mathlib/SetTheory/Nimber/Field.lean,Mathlib/Tactic/Linter/DirectoryDependency.lean,scripts/noshake.json 44 2 ['alreadydone', 'github-actions'] nobody
0-17982
4 hours ago
0-79625
22 hours ago
0-79669
22 hours
26845 kbuzzard
author:kbuzzard
chore: rename ValuativeTopology to IsValuativeTopology --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) It's a Prop but it involves topology so we have two conflicting naming conventions, namely the topologists' "`CompactSpace` is a perfectly fine name for a Prop and anyway we got used to it now" convention, and everyone else's `Is` convention. We're not used to this yet though so let's fix it. t-algebra
label:t-algebra$
41/9 Mathlib/RingTheory/Valuation/ValuativeRel.lean,Mathlib/Topology/Algebra/Valued/ValuativeRel.lean 2 3 ['Ruben-VandeVelde', 'github-actions', 'kbuzzard'] nobody
0-17860
4 hours ago
0-17870
4 hours ago
19-58052
19 days
24870 smmercuri
author:smmercuri
feat: `Field`, `FiniteDimensional` and `Algebra.IsSeparable` instances for `WithAbs` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-analysis 14/1 Mathlib/Analysis/Normed/Field/WithAbs.lean 1 1 ['github-actions'] fpvandoorn
assignee:fpvandoorn
0-17616
4 hours ago
79-54868
2 months ago
79-55009
79 days
22322 mariainesdff
author:mariainesdff
feat(RingTheory/DividedPowers/RatAlgebra): add definitions In this file we show that, for certain choices of a commutative (semi)ring `A` and an ideal `I` of `A`, the family of maps `ℕ → A → A` given by `fun n x ↦ x^n/n!` is a divided power structure on `I`. Co-authored-by: AntoineChambert-Loir --- - [x] depends on: #22237 - [x] depends on: #22239 - [x] depends on: #22240 - [x] depends on: #24439 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
324/2 Mathlib.lean,Mathlib/Data/Nat/Factorial/NatCast.lean,Mathlib/RingTheory/DividedPowers/RatAlgebra.lean 3 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] dagurtomas
assignee:dagurtomas
0-17616
4 hours ago
23-48446
23 days ago
30-79142
30 days
25974 scholzhannah
author:scholzhannah
feat(Topology/Compactness/CompactlyCoherentSpace): compact coherentification (k-ification) This PR defines the notion of turning an arbitrary topological space into a compactly coherent space. Compactly coherent spaces are commonly referred to as "compactly generated spaces" or "k-spaces" in the literature while the operation of turning a space into such as space is called the "k-ification". There are however three different notions that are described with this name. To disambiguate we use the names "compactly coherent space" and "compactcoherentification" here. See [this wikipedia page](https://en.wikipedia.org/wiki/Compactly_generated_space) for an explanation of these notions. This PR continues the work from #25318. Original PR: https://github.com/leanprover-community/mathlib4/pull/25318 Co-authored-by: Floris van Doorn large-import t-topology 175/5 Mathlib/Topology/Compactness/CompactlyCoherentSpace.lean 1 2 ['github-actions', 'scholzhannah'] ADedecker
assignee:ADedecker
0-17615
4 hours ago
46-6181
1 month ago
46-6229
46 days
26158 upobir
author:upobir
feat(NumberTheory/Divisors): add int divisors This PR continues the work from #25209. Original PR: https://github.com/leanprover-community/mathlib4/pull/25209 t-number-theory 101/4 Mathlib/NumberTheory/Divisors.lean 1 34 ['MichaelStollBayreuth', 'github-actions', 'upobir'] mariainesdff
assignee:mariainesdff
0-17614
4 hours ago
43-27586
1 month ago
43-27629
43 days
26272 ajirving
author:ajirving
feat(NumberTheory/LucasLehmer): prove converse direction to Lucas-Lehmer Proves the converse direction of the Lucas-Lehmer test, namely that the Lucas-Lehmer criterion is a necessary condition for a Mersenne prime. Adds a couple of examples of proving Mersenne numbers are composite using this. Proves that if `2^p-1` is prime then `p` is prime. --- * I wasn't sure how many examples to add given that there are many more Mersenne composites than primes. * There are a number of annoying coercions between different rings, any simplifications will be appreciated. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import new-contributor t-number-theory 226/5 Archive/Examples/MersennePrimes.lean,Mathlib/NumberTheory/LucasLehmer.lean 2 12 ['github-actions', 'kckennylau'] kbuzzard
assignee:kbuzzard
0-17613
4 hours ago
40-22302
1 month ago
40-22347
40 days
26277 AntoineChambert-Loir
author:AntoineChambert-Loir
feat(RingTheory/Congruence/Hom): prove basic isomorphisms theorems for ring congruences This file contains elementary definitions involving congruence relations and morphisms for semirings, rings, and algebras. * `RingCon.ker`: the kernel of a monoid homomorphism as a congruence relation * `RingCon.lift`, `RingCon.liftₐ`: the homomorphism / the algebra morphism on the quotient given that the congruence is in the kernel * `RingCon.map`, `RingCon.mapₐ`: homomorphism / algebra morphism from a smaller to a larger quotient * `RingCon.quotientKerEquivRangeS`, `RingCon.quotientKerEquivRange`, `RingCon.quotientKerEquivRangeₐ` : the first isomorphism theorem for semirings (using `RingHom.rangeS`), rings (using `RingHom.range`) and algebras (using `AlgHom.range`). * `RingCon.comapQuotientEquivRangeS`, `RingCon.comapQuotientEquivRange`, `RingCon.comapQuotientEquivRangeₐ` : the second isomorphism theorem for semirings (using `RingHom.rangeS`), rings (using `RingHom.range`) and algebras (using `AlgHom.range`). * `RingCon.quotientQuotientEquivQuotient`, `RingCon.quotientQuotientEquivQuotientₐ` : the third isomorphism theorem for semirings (or rings) and algebras It is an adaptation of what existed for multiplicative congruences (docs#Con) and is only useful for semirings which are not rings. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
555/2 Mathlib.lean,Mathlib/Algebra/Ring/Subsemiring/Basic.lean,Mathlib/Algebra/RingQuot.lean,Mathlib/RingTheory/Congruence/Basic.lean,Mathlib/RingTheory/Congruence/Defs.lean,Mathlib/RingTheory/Congruence/Hom.lean 6 1 ['github-actions'] joneugster
assignee:joneugster
0-17612
4 hours ago
39-85939
1 month ago
39-85986
39 days
26653 Hagb
author:Hagb
feat(RingTheory/Finiteness/Defs): span of a set is finitely generated iff generated by a finite subset --- This PR continues the work from #24651. Original PR: #24651. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 14/0 Mathlib/RingTheory/Finiteness/Defs.lean 1 1 ['github-actions'] jsm28
assignee:jsm28
0-17611
4 hours ago
27-20280
27 days ago
29-52478
29 days
26936 mariainesdff
author:mariainesdff
feat(RingTheory/DividedPowes/SubDPIdeal): complete lattice and quotients We show that sub-dp-ideals of a divided power ideal `I` of a ring `A` form a complete lattice under inclusion. Given an ideal `J` of `A`, we construct the divided power structure on the ideal `I(A⧸J)` of the quotient, provided that `I ⊓ J` is a sub-dp-ideal of `I`. Co-authored-by: @AntoineChambert-Loir --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-algebra
label:t-algebra$
314/16 Mathlib/LinearAlgebra/Span/Defs.lean,Mathlib/RingTheory/DividedPowers/SubDPIdeal.lean 2 1 ['github-actions'] joelriou
assignee:joelriou
0-17610
4 hours ago
23-25980
23 days ago
23-26031
23 days
26956 mariainesdff
author:mariainesdff
feat(RingTheory/DividedPowers/Basic): add divided power structure on pZp We construct a divided power structure on the ideal `(p) ⊆ ℤ_[p]`, given by the family of maps `fun n x ↦ x^n / n!`. Co-authored-by: @AntoineChambert-Loir --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 561/2 Mathlib.lean,Mathlib/Data/Nat/Factorial/NatCast.lean,Mathlib/RingTheory/DividedPowers/Padic.lean,Mathlib/RingTheory/DividedPowers/RatAlgebra.lean 4 1 ['github-actions'] mattrobball
assignee:mattrobball
0-17610
4 hours ago
22-42781
22 days ago
22-45123
22 days
27035 faenuccio
author:faenuccio
chore(IsManifold/Basic): replace continuity by aesop --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-differential-geometry easy 5/5 Mathlib/Geometry/Manifold/IsManifold/Basic.lean 1 3 ['faenuccio', 'fpvandoorn', 'github-actions'] sgouezel
assignee:sgouezel
0-17609
4 hours ago
20-18703
20 days ago
20-21590
20 days
27116 pechersky
author:pechersky
feat(Valued): FaithfulSMul to completion simplifies coercions and golfs existing instance --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-analysis t-number-theory
label:t-algebra$
16/6 Mathlib/RingTheory/DedekindDomain/AdicValuation.lean,Mathlib/Topology/Algebra/Valued/ValuedField.lean 2 1 ['github-actions'] mariainesdff
assignee:mariainesdff
0-17608
4 hours ago
18-57736
18 days ago
18-57737
18 days
27225 eric-wieser
author:eric-wieser
refactor(Tactic/Lift): deprecate the third with argument We already have a number of tactics where the clearing happens all the time, and you have to opt out with `id h`. This also fixes a bug where `lift z to Nat with n hn this_is_unused` would silently ignore `this_is_unused`. --- - [ ] depends on: #27223 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta 21/9 Mathlib/Tactic/Lift.lean,MathlibTest/lift.lean 2 5 ['JovanGerb', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'vihdzp'] JovanGerb
assignee:JovanGerb
0-17607
4 hours ago
14-81926
14 days ago
15-8006
15 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/) new-contributor t-algebra
label:t-algebra$
106/0 Mathlib/GroupTheory/DoubleCoset.lean 1 1 ['github-actions'] mariainesdff
assignee:mariainesdff
0-17607
4 hours ago
15-21359
15 days ago
15-21409
15 days
27248 kckennylau
author:kckennylau
chore: remove `suppress_compilation` from Mathlib.Algebra.Category.Ring.Constructions --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra easy
label:t-algebra$
2/4 Mathlib/Algebra/Category/Ring/Constructions.lean 1 4 ['github-actions', 'grunweg', 'leanprover-bot'] chrisflav
assignee:chrisflav
0-17606
4 hours ago
14-36412
14 days ago
14-36460
14 days
27255 Louddy
author:Louddy
feat(SkewMonoidAlgebra): coeff_mul lemmas Add lemmas regarding the interaction of multiplication and the `SkewMonoidAlgebra.coeff`. Co-authored-by: María Inés de Frutos Fernández <[mariaines.dff@gmail.com](mailto:mariaines.dff@gmail.com)> --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
124/0 Mathlib/Algebra/SkewMonoidAlgebra/Basic.lean 1 1 ['github-actions'] chrisflav
assignee:chrisflav
0-17605
4 hours ago
14-25747
14 days ago
14-25738
14 days
27368 alreadydone
author:alreadydone
feat(FieldTheory/Finite): minimal polynomial of Frobenius for the normal basis theorem at *Formalizing Class Field Theory* --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
37/5 Mathlib/Algebra/Algebra/Equiv.lean,Mathlib/Algebra/Algebra/Hom.lean,Mathlib/FieldTheory/Finite/Basic.lean,Mathlib/FieldTheory/Minpoly/Basic.lean 4 6 ['alreadydone', 'github-actions', 'kckennylau'] riccardobrasca
assignee:riccardobrasca
0-17604
4 hours ago
7-27130
7 days ago
7-79303
7 days
27461 IvanRenison
author:IvanRenison
feat(Combinatorics/SimpleGraph/Paths): add lemma `SimpleGraph.Walk.IsPath.mem_support_iff_exists_append` This contribution was created as part of the Utrecht Summerschool "Formalizing Mathematics in Lean" in July 2025. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics 14/0 Mathlib/Combinatorics/SimpleGraph/Paths.lean 1 1 ['github-actions'] awainverse
assignee:awainverse
0-17603
4 hours ago
7-41447
7 days ago
7-41491
7 days
27840 CBirkbeck
author:CBirkbeck
feat(NumberTheory/ModularForms/EisensteinSeries): define gammaSetN --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-number-theory 75/1 Mathlib/NumberTheory/ModularForms/EisensteinSeries/Defs.lean 1 1 ['github-actions'] nobody
0-17075
4 hours ago
0-17785
4 hours ago
0-17827
4 hours
27743 alreadydone
author:alreadydone
feat(NumberTheory): Frobenius number exists, ℕ is Noetherian semiring & Sylver coinage + The Frobenius number of a set of natural numbers exist iff the set has gcd 1 and doesn't contain 1. + All additive submonoids (= ideals) of ℕ are finitely generated. + The game of Sylver coinage always terminates. This is the outcome of a course project at Heidelberg University: [matematiflo.github.io/CompAssistedMath2025](https://matematiflo.github.io/CompAssistedMath2025/) Co-authored-by: Daniel Buth @greymatter8 Co-authored-by: Sebastian Meier @SebastianMeierUni --- FrobeniusNumber is a leaf file so I think doubling its imports is okay. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-algebra t-combinatorics t-number-theory
label:t-algebra$
259/28 Mathlib/Data/Set/Finite/Basic.lean,Mathlib/LinearAlgebra/FreeModule/PID.lean,Mathlib/NumberTheory/FrobeniusNumber.lean,Mathlib/RingTheory/Ideal/NatInt.lean,Mathlib/RingTheory/PrincipalIdealDomain.lean 5 2 ['github-actions', 'vihdzp'] nobody
0-16797
4 hours ago
1-12395
1 day ago
1-37996
1 day
26981 JovanGerb
author:JovanGerb
chore: golf using `grw` This PR cleans up some proofs using `grw`. It also tags a few lemmas with `@[gcongr]` that were required for the proofs. --- - [ ] depends on: #26907 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import 179/202 Archive/Wiedijk100Theorems/CubingACube.lean,Mathlib/Algebra/Category/ModuleCat/Topology/Basic.lean,Mathlib/Algebra/Group/Subgroup/Basic.lean,Mathlib/Algebra/Group/Subgroup/Map.lean,Mathlib/Algebra/Lie/Engel.lean,Mathlib/Algebra/Lie/IdealOperations.lean,Mathlib/Algebra/Module/Submodule/IterateMapComap.lean,Mathlib/Algebra/Order/Archimedean/Basic.lean,Mathlib/Algebra/Order/CauSeq/BigOperators.lean,Mathlib/Algebra/Order/Field/Basic.lean,Mathlib/Algebra/Order/Group/Multiset.lean,Mathlib/Algebra/Order/Kleene.lean,Mathlib/Algebra/Order/Rearrangement.lean,Mathlib/Algebra/Order/Ring/Unbundled/Basic.lean,Mathlib/Analysis/BoxIntegral/Integrability.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Isometric.lean,Mathlib/Analysis/Calculus/ContDiff/Bounds.lean,Mathlib/Analysis/Convex/Gauge.lean,Mathlib/Analysis/Convex/Slope.lean,Mathlib/Analysis/Distribution/SchwartzSpace.lean,Mathlib/Analysis/Normed/Affine/AddTorsor.lean,Mathlib/Analysis/Normed/Order/UpperLower.lean,Mathlib/Analysis/NormedSpace/OperatorNorm/NNNorm.lean,Mathlib/Analysis/Oscillation.lean,Mathlib/Analysis/SpecialFunctions/Pow/NNReal.lean,Mathlib/Combinatorics/Additive/AP/Three/Behrend.lean,Mathlib/Combinatorics/Hall/Finite.lean,Mathlib/Data/NNReal/Defs.lean,Mathlib/Data/Real/Cardinality.lean,Mathlib/Dynamics/Ergodic/MeasurePreserving.lean,Mathlib/FieldTheory/IntermediateField/Adjoin/Basic.lean,Mathlib/LinearAlgebra/AffineSpace/Ordered.lean,Mathlib/MeasureTheory/Covering/LiminfLimsup.lean,Mathlib/MeasureTheory/Integral/Bochner/Basic.lean,Mathlib/MeasureTheory/Integral/Bochner/Set.lean,Mathlib/MeasureTheory/Integral/Bochner/VitaliCaratheodory.lean,Mathlib/MeasureTheory/Integral/DominatedConvergence.lean,Mathlib/MeasureTheory/Integral/IntegralEqImproper.lean,Mathlib/MeasureTheory/Measure/Content.lean,Mathlib/MeasureTheory/Measure/EverywherePos.lean,Mathlib/MeasureTheory/Measure/IntegralCharFun.lean,Mathlib/MeasureTheory/Measure/Lebesgue/Basic.lean,Mathlib/MeasureTheory/Measure/Stieltjes.lean,Mathlib/MeasureTheory/OuterMeasure/Caratheodory.lean,Mathlib/MeasureTheory/OuterMeasure/Induced.lean,Mathlib/MeasureTheory/OuterMeasure/OfFunction.lean,Mathlib/NumberTheory/ClassNumber/AdmissibleCardPowDegree.lean,Mathlib/NumberTheory/FLT/Polynomial.lean,Mathlib/NumberTheory/ModularForms/JacobiTheta/TwoVariable.lean,Mathlib/NumberTheory/Transcendental/Lindemann/AnalyticalPart.lean,Mathlib/Order/Basic.lean,Mathlib/Order/BooleanAlgebra/Basic.lean,Mathlib/Order/Closure.lean,Mathlib/Order/ConditionallyCompleteLattice/Basic.lean,Mathlib/Order/Height.lean,Mathlib/Order/Interval/Set/Monotone.lean,Mathlib/Order/Monotone/Extension.lean,Mathlib/Order/PrimeSeparator.lean,Mathlib/Probability/Martingale/Upcrossing.lean,Mathlib/Probability/Process/HittingTime.lean,Mathlib/RingTheory/Ideal/Operations.lean,Mathlib/RingTheory/MvPowerSeries/PiTopology.lean,Mathlib/RingTheory/Polynomial/Basic.lean,Mathlib/SetTheory/Cardinal/Arithmetic.lean,Mathlib/SetTheory/Cardinal/Ordinal.lean,Mathlib/SetTheory/Ordinal/Basic.lean,Mathlib/SetTheory/Ordinal/Enum.lean,Mathlib/SetTheory/Ordinal/FixedPointApproximants.lean,Mathlib/Topology/Maps/Basic.lean,Mathlib/Topology/MetricSpace/Holder.lean,Mathlib/Topology/MetricSpace/Kuratowski.lean,Mathlib/Topology/MetricSpace/Thickening.lean,Mathlib/Topology/NhdsSet.lean,Mathlib/Topology/Order.lean 74 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
0-14673
4 hours ago
0-83054
23 hours ago
1-2089
1 day
27400 dleijnse
author:dleijnse
feat: define geometrically reduced algebras Define geometrically reduced algebras, and prove that if all finitely generated subalgebras of an algebra `A` are geometrically reduced, then `A` is geometrically reduced. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra
label:t-algebra$
111/0 Mathlib.lean,Mathlib/RingTheory/Nilpotent/GeometricallyReduced.lean 2 23 ['dleijnse', 'github-actions', 'kckennylau'] nobody
0-14497
4 hours ago
9-6574
9 days ago
9-6619
9 days
27839 CBirkbeck
author:CBirkbeck
feat(NumberTheory/ModularForms/EisensteinSeries): define normalised Eisenstein series in preparation for giving their q-expansions. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-number-theory 11/0 Mathlib/NumberTheory/ModularForms/EisensteinSeries/Basic.lean 1 1 ['github-actions'] nobody
0-14387
3 hours ago
0-18257
5 hours ago
0-18306
5 hours
27843 JovanGerb
author:JovanGerb
feat(Data/Nat/Basic): `Nat.sub_le_sub` This PR adds the missing lemma `Nat.sub_le_sub`, because the usual `sub_le_sub` doesn't work for `Nat`. TODO: use `gcongr`/`grw` using this new lemma. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data 4/0 Mathlib/Data/Nat/Basic.lean 1 1 ['github-actions'] nobody
0-13722
3 hours ago
0-13745
3 hours ago
0-13791
3 hours
26036 joelriou
author:joelriou
feat(CategoryTheory/Functor): pointwise right derived functors This PR introduces pointwise right derived functors as particular cases of pointwise left Kan extensions. --- This PR continues the work from #22490. Original PR: https://github.com/leanprover-community/mathlib4/pull/22490 maintainer-merge t-category-theory 169/0 Mathlib.lean,Mathlib/CategoryTheory/Functor/Derived/PointwiseRightDerived.lean 2 13 ['github-actions', 'joelriou', 'robin-carlier'] robin-carlier
assignee:robin-carlier
0-12990
3 hours ago
0-41405
11 hours ago
44-65753
44 days
27457 grunweg
author:grunweg
feat(LocallyIntegrable): generalise the first half of the file to enorms --- This is not exhaustive; all `smul` lemmas can also be generalised (assuming suitable typeclasses). That will happen in a separate PR. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) carleson maintainer-merge t-measure-probability 90/48 Mathlib/MeasureTheory/Function/LocallyIntegrable.lean,Mathlib/MeasureTheory/Integral/IntegrableOn.lean 2 11 ['YaelDillies', 'github-actions', 'grunweg'] EtienneC30
assignee:EtienneC30
0-12870
3 hours ago
0-12870
3 hours ago
7-50585
7 days
27846 euprunin
author:euprunin
chore(Algebra/Group): golf `range_eq_image_or_of_mulSupport_subset` using `grind` maintainer-merge t-algebra
label:t-algebra$
1/4 Mathlib/Algebra/Group/Support.lean 1 2 ['github-actions', 'grunweg'] nobody
0-11549
3 hours ago
0-11549
3 hours ago
0-13488
3 hours
27810 euprunin
author:euprunin
chore(Algebra/BigOperators): golf `prod_list_map_count` using `grind [Finset.prod_congr]` maintainer-merge t-algebra
label:t-algebra$
1/5 Mathlib/Algebra/BigOperators/Group/Finset/Basic.lean 1 2 ['github-actions', 'grunweg'] nobody
0-11140
3 hours ago
0-11140
3 hours ago
0-42240
11 hours
27811 euprunin
author:euprunin
chore(Algebra/PresentedMonoid): golf `ext` using `grind [Set.eqOn_range]` maintainer-merge t-algebra
label:t-algebra$
1/4 Mathlib/Algebra/PresentedMonoid/Basic.lean 1 2 ['github-actions', 'grunweg'] nobody
0-11127
3 hours ago
0-11127
3 hours ago
0-42156
11 hours
27808 euprunin
author:euprunin
chore(Algebra): golf `surj_of_gcd_domain`, `toCommMonoid_injective`, `f_eq`, `eq_top_of_invtSubmodule_ne_bot` and `dvd_mul_sub_mul_mul_left_of_dvd` using `grind` maintainer-merge t-algebra
label:t-algebra$
5/13 Mathlib/Algebra/GCDMonoid/IntegrallyClosed.lean,Mathlib/Algebra/Group/Ext.lean,Mathlib/Algebra/Homology/Embedding/HomEquiv.lean,Mathlib/Algebra/Lie/Weights/RootSystem.lean,Mathlib/Algebra/Ring/Divisibility/Lemmas.lean 5 2 ['github-actions', 'grunweg'] nobody
0-11113
3 hours ago
0-11113
3 hours ago
0-42482
11 hours
27663 ShreckYe
author:ShreckYe
feat(Analysis/SpecialFunctions/Trigonometric/Basic): add the duals named `cos_eq_zero_iff_sin_eq` for the theorems named `sin_eq_zero_iff_cos_eq` in both real and complex cases Similar to #27622. These seem missing for cosine case. I simplified the proofs adapted from `sin_eq_zero_iff_cos_eq` using `simp` compared to the original way of constructing the remaining goal explictly using `exact`. If needed, I can simplify the proofs of the 2 `sin_eq_zero_iff_cos_eq`s too. new-contributor t-analysis easy 8/0 Mathlib/Analysis/SpecialFunctions/Trigonometric/Basic.lean 1 6 ['ShreckYe', 'github-actions', 'themathqueen'] nobody
0-9927
2 hours ago
1-38671
1 day ago
2-69922
2 days
27848 dupuisf
author:dupuisf
feat: mathlib instance for `Lean.Grind.LinearOrder` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order 3/0 Mathlib/Order/Defs/LinearOrder.lean 1 1 ['github-actions'] nobody
0-8979
2 hours ago
0-8979
2 hours ago
0-9028
2 hours
27699 mans0954
author:mans0954
refactor(Analysis/Normed/Module/Dual): Abbrev for topological dual The concept of a topological dual can be defined whenever `E →L[𝕜] 𝕜` makes sense. Discussion: https://github.com/leanprover-community/mathlib4/pull/26345/files#r2234132483 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 130/124 Mathlib/Analysis/InnerProductSpace/Adjoint.lean,Mathlib/Analysis/InnerProductSpace/Dual.lean,Mathlib/Analysis/Normed/Module/Dual.lean,Mathlib/Analysis/Normed/Module/WeakDual.lean,Mathlib/Analysis/VonNeumannAlgebra/Basic.lean,Mathlib/MeasureTheory/Function/AEEqOfIntegral.lean,Mathlib/MeasureTheory/Measure/CharacteristicFunction.lean,Mathlib/MeasureTheory/Measure/IntegralCharFun.lean,Mathlib/Probability/Distributions/Gaussian/Basic.lean,Mathlib/Probability/Moments/CovarianceBilin.lean,Mathlib/Topology/Algebra/Module/LinearMap.lean,docs/overview.yaml,docs/undergrad.yaml 13 21 ['eric-wieser', 'github-actions', 'j-loreaux', 'mans0954', 'themathqueen'] nobody
0-7943
2 hours ago
2-2242
2 days ago
2-4879
2 days
27845 themathqueen
author:themathqueen
feat(Analysis/InnerProductSpace/Adjoint): some API for `innerSL` In [bra-ket notation](https://en.wikipedia.org/wiki/Bra–ket_notation), these are: - $\langle x|^\dagger=|x\rangle$, - $f\circ|x\rangle=|f(x)\rangle$, - $\langle x|\circ f=\langle f^\dagger(x)|$, where $\langle x|$ is `innerSL _ x`, and $|x\rangle$ is `(lsmul _ _).flip x`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis 19/0 Mathlib/Analysis/InnerProductSpace/Adjoint.lean,Mathlib/Analysis/NormedSpace/OperatorNorm/Mul.lean 2 1 ['github-actions'] nobody
0-4736
1 hour ago
0-13574
3 hours ago
0-13625
3 hours
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/) t-algebra
label:t-algebra$
27/0 Mathlib/RingTheory/Valuation/Basic.lean 1 7 ['JovanGerb', 'github-actions', 'pechersky', 'wwylele'] nobody
0-4125
1 hour ago
7-76710
7 days ago
7-76758
7 days
27835 edegeltje
author:edegeltje
feat(Tactic): ring modulo a given characteristic (resurrection of #10765, attempt two) This used to be #10765 by Anne Baanen before the great forkening. > This PR extends the `ring` tactic with a new config argument `char` which will try to reduce all constant terms modulo the given characteristic. This allows `ring` to prove e.g. `(x + y)^3 = x^3 + y^3` in characteristic 3. This is a simpler and faster way to do so than what we had before: `repeat { ring; reduce_mod_char }` becomes `ring (config := { char := 3 })`. > > The first step is to split off the required `CharP` definitions, since `Mathlib.Algebra.CharP.Basic` already requires the `ring` tactic. > > To perform the reduction modulo the given characteristic, I implemented `reduceCast` which reduces a raw integer, and wrapped it in `reduceResult` that takes a `NormNum.Result` for easy use. We need to pass through quite a few parameters into `reduceResult` so maybe it's worth defining a structure, or reusing `Cache` for this. > > Then it's basically a case of replacing every place where `ring` constructs a numeral with a call to `reduceResult`. > > Limitations: > > * `ring` doesn't attempt to detect the characteristic by itself, you need to pass it in explicitly. Trying to infer a `CharP` instance at each point sounds quite expensive. > > * Since the support for `%` in `NormNum` only exists for integers, I implemented the reduction only when a `Ring` instance is available. It is still sound in the semiring case, just not complete. > > * We could optimize exponentiation in the specific case where the characteristic `p` is a prime that divides the exponent `n`: `(x + y)^n = x^n + y^n`. I'll leave that to future work. > --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) migrated-from-branch large-import t-meta 309/134 Mathlib/LinearAlgebra/Eigenspace/Basic.lean,Mathlib/RingTheory/MvPolynomial/Basic.lean,Mathlib/Tactic/LinearCombination.lean,Mathlib/Tactic/Module.lean,Mathlib/Tactic/Polyrith.lean,Mathlib/Tactic/Ring/Basic.lean,Mathlib/Tactic/Ring/Compare.lean,Mathlib/Tactic/Ring/RingNF.lean,MathlibTest/ring_compare.lean,MathlibTest/ring_mod_char.lean 10 2 ['edegeltje', 'github-actions'] joneugster
assignee:joneugster
0-2067
34 minutes ago
0-2274
37 minutes ago
0-2285
38 minutes
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/) t-algebra
label:t-algebra$
35/0 Mathlib/Algebra/QuadraticDiscriminant.lean 1 4 ['github-actions', 'tb65536', 'upobir'] chrisflav
assignee:chrisflav
0-1445
24 minutes ago
43-27234
1 month ago
43-27277
43 days
27362 101damnations
author:101damnations
feat(RepresentationTheory): add the norm map Given a representation `A` of a finite group `G`, `A.norm` is the representation morphism `A ⟶ A` defined by `x ↦ ∑ A.ρ g x` for `g` in `G`. We define this and prove related lemmas. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) maintainer-merge t-algebra
label:t-algebra$
151/0 Mathlib/Algebra/BigOperators/Fin.lean,Mathlib/RepresentationTheory/Basic.lean,Mathlib/RepresentationTheory/Rep.lean 3 7 ['101damnations', 'github-actions', 'kbuzzard'] nobody
0-999
16 minutes ago
6-1908
6 days ago
9-84977
9 days
27847 euprunin
author:euprunin
chore(Algebra): avoid duplicating proofs by reusing existing theorems or lemmas t-algebra
label:t-algebra$
9/36 Mathlib/Algebra/Homology/Embedding/Extend.lean,Mathlib/Algebra/MvPolynomial/Rename.lean,Mathlib/Algebra/Order/Group/Abs.lean,Mathlib/Algebra/Order/Ring/Unbundled/Rat.lean,Mathlib/Algebra/Polynomial/Degree/Lemmas.lean,Mathlib/Algebra/Polynomial/Monic.lean 6 6 ['github-actions', 'grunweg', 'kbuzzard'] nobody
0-781
13 minutes ago
0-12433
3 hours ago
0-12485
3 hours
24527 matthewjasper
author:matthewjasper
feat(Topology/Algebra/Module): Add more theorems for IsModuleTopology Add theorems that surjective linear maps to the module topology are open. Add IsModuleTopology instance for quotients. Add IsModuleTopology instance for finite dimensional T2 vector spaces over a complete normed field and use it to shorten some proofs. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra t-topology
label:t-algebra$
52/26 Mathlib/Analysis/Fourier/AddCircleMulti.lean,Mathlib/Analysis/RCLike/Lemmas.lean,Mathlib/Topology/Algebra/Module/FiniteDimension.lean,Mathlib/Topology/Algebra/Module/ModuleTopology.lean 4 8 ['erdOne', 'github-actions', 'matthewjasper', 'ocfnash', 'riccardobrasca'] ocfnash
assignee:ocfnash
0-387
6 minutes ago
90-35968
2 months ago
92-4263
92 days

New contributors' PRs on the review queue

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
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/) new-contributor t-combinatorics 187/0 Mathlib.lean,Mathlib/Combinatorics/SimpleGraph/Cycle.lean 2 29 ['IvanRenison', 'github-actions'] kmill
assignee:kmill
71-73849
2 months ago
99-71406
3 months ago
99-71456
99 days
25858 themathqueen
author:themathqueen
feat(RingTheory/Coalgebra/MulOpposite): coalgebra instance for MulOpposite Adding an instance for `Aᵐᵒᵖ` being an `R`-coalgebra when `A` is. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra
label:t-algebra$
112/0 Mathlib.lean,Mathlib/RingTheory/Coalgebra/MulOpposite.lean 2 1 ['github-actions'] nobody
43-85580
1 month ago
48-30979
1 month ago
48-31022
48 days
26301 Ivan-Sergeyev
author:Ivan-Sergeyev
feat(LinearAlgebra/Matrix/Determinant/TotallyUnimodular): Empty matrices are totally unimodular. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra
label:t-algebra$
15/0 Mathlib/LinearAlgebra/Matrix/Determinant/TotallyUnimodular.lean 1 1 ['github-actions'] nobody
39-28860
1 month ago
39-28870
1 month ago
39-28913
39 days
26462 PSchwahn
author:PSchwahn
feat(LinearAlgebra/Projection): add results about inverse of `Submodule.prodEquivOfIsCompl` Add two theorems `Submodule.prodEquivOfIsCompl_symm_apply` and `Submodule.prodEquivOfIsCompl_symm_add`, which are API for `Submodule.prodEquivOfIsCompl`. We believe these theorems are useful; for example, we have used their statements in a [classification formalization project](https://github.com/LieLean/LowDimSolvClassification). I am not sure whether the `prodEquivOfIsCompl_symm_apply` theorem should be tagged with `@[simp]`; this might lead to confluence issues. Opinions are welcome! Co-authored by: - [Viviana del Barco](https://github.com/vdelbarc) - [Gustavo Infanti](https://github.com/GuQOliveira) - [Exequiel Rivas](https://github.com/erivas) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra
label:t-algebra$
9/0 Mathlib/LinearAlgebra/Projection.lean 1 5 ['PSchwahn', 'github-actions', 'kckennylau'] nobody
33-80619
1 month ago
35-66253
1 month ago
35-66377
35 days
23986 ShouxinZhang
author:ShouxinZhang
feat(FieldTheory/RatFunc): add RatFunc.toFractionRingAlgEquiv --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra
label:t-algebra$
13/0 Mathlib/FieldTheory/RatFunc/Basic.lean 1 32 ['ShouxinZhang', 'eric-wieser', 'github-actions', 'joneugster', 'kckennylau', 'plp127'] nobody
29-75617
29 days ago
32-2073
1 month ago
110-65010
110 days
26710 metakunt
author:metakunt
feat (Data/Nat/Digits/Lemmas): Add digits_getD Adds digits_getD, an explicit computation of the i-th digits of n in base b representation. t-data new-contributor 64/0 Mathlib/Data/Nat/Digits/Lemmas.lean 1 1 ['github-actions'] nobody
28-77564
28 days ago
28-77695
28 days ago
28-77746
28 days
26814 KiringYJ
author:KiringYJ
feat(MeasureTheory): expose `m.SigmaAlgebra` and `IsSigmaAlgebra` (New PR opened because I mis-clicked “Merge” on the previous branch and had to revert it.) This PR introduces a lightweight API for treating the σ‑algebra of a `MeasurableSpace` as a plain `Set (Set α)`, plus a semantic predicate `IsSigmaAlgebra` and small bridges between bundled and un‑bundled views. #### Motivation The immediate goal is to prepare for a formalization of the **monotone class theorem**. With `m.SigmaAlgebra` and the `IsSigmaAlgebra` predicate, one can state the theorem as a clean equality of families of sets, e.g. ```lean SigmaAlgebra.generateFrom G = MonotoneClass.generateFrom G ``` rather than the more cumbersome phrasing "`s` is measurable ↔ `s` belongs to the smallest monotone class containing `G`". The helpers in this PR make those equalities ergonomic and reusable. #### What’s new - **`m.SigmaAlgebra`** – the collection of all `m`‑measurable sets, exposed as a value of type `Set (Set α)`. Lets you write `s ∈ m.SigmaAlgebra` instead of `MeasurableSet[m] s`. - **`IsSigmaAlgebra F`** – predicate saying that a family of sets `A` is already a σ‑algebra, defined by `(generateFrom F).SigmaAlgebra = F`. - **`generateFrom_sigmaAlgebra_eq`** – idempotence lemma `generateFrom m.SigmaAlgebra = m` (`@[simp]`). - Boolean‑algebra instance on `m.SigmaAlgebra` (alias of the existing subtype instance). - Helper lemmas: - `Subtype.mem_sigma` – bundled measurable set ∈ `m.SigmaAlgebra`. - `Set.toMeasurableSubtype` – wrap a membership proof into the subtype. #### House‑keeping - Removed two obsolete `noncomputable` keywords from `Mathlib/MeasureTheory/MeasurablyGenerated.lean`; the affected instances are now computable. #### Notes - **No breaking changes**: the new definitions are additive; existing code continues to compile unchanged. - **No dependencies on other PRs**: this patch is self‑contained. new-contributor t-measure-probability 86/3 Mathlib.lean,Mathlib/MeasureTheory/MeasurableSpace/MeasurablyGenerated.lean,Mathlib/MeasureTheory/MeasurableSpace/SigmaAlgebra.lean 3 1 ['github-actions'] nobody
22-56765
22 days ago
26-45734
26 days ago
26-45778
26 days
26881 emo916math
author:emo916math
feat(Analysis/Calculus/Deriv/Star) A formula for `deriv (conj ∘ f ∘ conj)` Added a lemma that `deriv (conj ∘ f ∘ conj) = conj ∘ deriv f ∘ conj`, proved by cases on whether the derivative mathematically exists or not. This PR replaces [#26805](https://github.com/leanprover-community/mathlib4/pull/26805); see discussion there. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-analysis 50/2 Mathlib/Analysis/Calculus/Deriv/Star.lean 1 7 ['emo916math', 'github-actions', 'kckennylau'] nobody
22-8646
22 days ago
25-5684
25 days ago
25-5728
25 days
27000 gasparattila
author:gasparattila
feat(Analysis/Normed/Group/Quotient): isometric versions of isomorphisms This PR adds an isometric version of the third isomorphism theorem for groups and modules. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import new-contributor t-analysis 49/2 Mathlib/Analysis/Normed/Group/Quotient.lean 1 1 ['github-actions'] nobody
21-27046
21 days ago
21-27048
21 days ago
21-27100
21 days
27200 rotarc75
author:rotarc75
feat(RingTheory/Ideal): oka predicates over ideals This PR introduces the notion of Oka predicates over the ideals of a ring. We usually speak of [Oka families](https://stacks.math.columbia.edu/tag/05K9) but predicates seemed more in line with mathlib's conventions. Currently this notions isn't used anywhere but we plan to make an other PR that proves that is all prime ideals of a ring are finitely generated, then this ring is Noetherian. We can also use Oka predicates to simplify the existing proof of [`IsPrincipalIdealRing.of_prime`](https://leanprover-community.github.io/mathlib4_docs/Mathlib/RingTheory/PrincipalIdealDomainOfPrime.html#IsPrincipalIdealRing.of_prime). Co-authored-by: Anthony Fernandes --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra
label:t-algebra$
53/0 Mathlib.lean,Mathlib/RingTheory/Ideal/Oka.lean 2 1 ['github-actions'] nobody
16-38859
16 days ago
16-38859
16 days ago
16-39758
16 days
27226 xcloudyunx
author:xcloudyunx
feat(Combinatorics/SimpleGraph): Add Subgraph.inclusion_edge_apply_coe and inclusion_edgeSet_apply_coe This PR continues the work from #25248. Original PR: https://github.com/leanprover-community/mathlib4/pull/25248 new-contributor t-combinatorics 14/0 Mathlib/Combinatorics/SimpleGraph/Subgraph.lean 1 1 ['github-actions'] nobody
15-72397
15 days ago
15-73816
15 days ago
15-73872
15 days
27245 rirarika
author:rirarika
MvPolynomial.Irreducible --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra
label:t-algebra$
88/0 Mathlib.lean,Mathlib/Algebra/MvPolynomial/Irreducible.lean 2 3 ['alreadydone', 'github-actions', 'mbkybky'] nobody
14-22675
14 days ago
14-49164
14 days ago
14-49207
14 days
27261 Sebi-Kumar
author:Sebi-Kumar
feat(Topology): add definition for subpaths Define subpaths as restrictions of paths to subintervals, reparameterized to have domain `[0, 1]` and possibly with a reverse of direction. Prove their basic properties. This serves as an alternative to `Path.truncate` which is useful for the explicit construction of certain homotopies, in particular regarding the concatenation of subpaths. --- To provide additional context, this is my first time contributing to Mathlib, and I am doing so as a part of the Fields Undergraduate Summer Research Program hosted at Western University. My intention for this file is for it to be used when proving that the fundamental group of the sphere is trivial (following the proof from Hatcher's "Algebraic Topology"). [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-topology 148/0 Mathlib.lean,Mathlib/Topology/Subpath.lean 2 1 ['github-actions'] nobody
14-1698
14 days ago
14-12329
14 days ago
14-12376
14 days
26880 agjftucker
author:agjftucker
feat(Calculus/FDeriv/Partial): `hasStrictFDerivAt_uncurry_coprod` concerning partial derivatives Confident that other contributions will follow (e.g. #26300), I begin this file with only the result needed to apply the implicit function theorem to a curried function. --- - [x] depends on: #26742 [This dependency is very slight.] [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor 126/0 Mathlib.lean,Mathlib/Analysis/Calculus/FDeriv/Partial.lean 2 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
13-5557
13 days ago
13-5557
13 days ago
16-83137
16 days
27242 hugh-fox
author:hugh-fox
feat: add Gauss-like formula for sums of digit sums Adds `sum_digit_sum_base_pow_eq` to show a Gauss-like formula across sums of digit sums. This relies on an additional two simp lemmas, named `digits_sum_eq_self`, `digits_sum_base_mul_cancel`. Lastly, includes a specialization (which is a good bit simpler than the general formula) to base 10 named `sum_digit_sum_ten_pow_eq`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-data new-contributor 113/0 Mathlib/Data/Nat/Digits/Lemmas.lean 1 5 ['github-actions', 'hugh-fox', 'kckennylau'] nobody
13-4460
13 days ago
14-68238
14 days ago
14-68284
14 days
27082 staroperator
author:staroperator
feat(Order/WellFoundedSet): add `Set.IsPWO.exists_le_minimal`, `Set.IsPWO.exists_minimal`, `Set.IsPWO.exists_minimalFor` which are the `IsPWO` version of `exists_minimal_le_of_wellFoundedLT` and others. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-order 22/0 Mathlib/Order/WellFoundedSet.lean 1 4 ['alreadydone', 'github-actions', 'staroperator'] nobody
10-67169
10 days ago
19-16583
19 days ago
19-16628
19 days
27357 jcreedcmu
author:jcreedcmu
feat(Algebra/Module/Submodule): add `submoduleMap` for isometries Per [discussion on Zulip](https://leanprover.zulipchat.com/#narrow/channel/217875-Is-there-code-for-X.3F/topic/Analog.20of.20LinearEquiv.2EsubmoduleMap.20for.20AffineIsometryEquiv.3F), add a version of `.submoduleMap` for `LinearIsometry` and `LinearIsometryEquiv` by analogy with `LinearMap.submoduleMap` and `LinearEquiv.submoduleMap`. --- new-contributor t-algebra
label:t-algebra$
56/0 Mathlib.lean,Mathlib/Analysis/Normed/Operator/LinearIsometrySubmoduleMap.lean 2 12 ['Ruben-VandeVelde', 'eric-wieser', 'github-actions', 'jcreedcmu'] nobody
9-84952
9 days ago
10-3735
10 days ago
10-3786
10 days
27040 Scarlett-le
author:Scarlett-le
feat(Geometry/Euclidean/Sphere/Power): add power of a point theorems Add the definition of power of a point and fundamental theorems relating point positions to intersection distances: * `Sphere.power`: The power of a point with respect to a sphere, defined as the square of the distance from the point to the center minus the square of the radius. * `Sphere.power_eq_zero_iff_mem_sphere`: A point lies on the sphere if and only if its power is zero. * `Sphere.power_pos_iff_dist_center_gt_radius`: The power is positive if and only if the point is outside the sphere. * `Sphere.power_neg_iff_dist_center_lt_radius`: The power is negative if and only if the point is inside the sphere. * `Sphere.mul_dist_eq_power_of_dist_center_gt_radius`: For external points, the product of intersection distances equals the power. * `Sphere.mul_dist_eq_neg_power_of_dist_center_lt_radius`: For internal points, the product equals the negative power. * `Sphere.mul_dist_eq_abs_power`: General form relating intersection distance products to absolute power. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-euclidean-geometry 138/1 Mathlib/Geometry/Euclidean/Sphere/Power.lean 1 3 ['alreadydone', 'github-actions'] jsm28
assignee:jsm28
9-42756
9 days ago
20-10223
20 days ago
20-10763
20 days
26783 matthewjasper
author:matthewjasper
feat(RingTheory/Flat): Add theorems relating Submodule.torsion and Module.Flat Co-authored-by: Kevin Buzzard --- This PR continues the work from #25334. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) FLT new-contributor t-algebra
label:t-algebra$
205/0 Mathlib.lean,Mathlib/Algebra/Algebra/Bilinear.lean,Mathlib/Algebra/Module/LocalizedModule/Basic.lean,Mathlib/RingTheory/Flat/TorsionFree.lean,Mathlib/RingTheory/Ideal/IsPrincipal.lean 5 1 ['github-actions'] nobody
8-1531
8 days ago
27-33973
27 days ago
27-34001
27 days
27472 guelmi94
author:guelmi94
feat(Combinatorics/SimpleGraph/Walk): add lemma `support_injective` This contribution was created as part of the Utrecht Summerschool "Formalizing Mathematics in Lean" in July 2025. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-combinatorics 3/0 Mathlib/Combinatorics/SimpleGraph/Walk.lean 1 1 ['github-actions'] nobody
7-25313
7 days ago
7-25316
7 days ago
7-25364
7 days
25951 themathqueen
author:themathqueen
feat(Analysis/InnerProductSpace/MulOpposite): defines the inner product on opposite spaces This pr defines the inner product on opposite spaces. - [x] depends on: #25949 Motivation for having the inner product structure on the opposite: One application comes up in non-commutative graphs, which are defined on a finite-dimensional C*-algebra with a faithful and positive functional (a Hilbert space structure can be induced by the defined faithful and positive functional (will be added to a pr soon)). For example, we'd need the Hilbert space structure to be defined on the opposite space to define the isomorphism: `(A →ₗ[ℂ] B) ≃ₗ[ℂ] TensorProduct ℂ B Aᵐᵒᵖ`, where `A`, `B` are again finite-dimensional C*-algebras with faithful and positive functionals. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor 71/0 Mathlib.lean,Mathlib/Analysis/InnerProductSpace/MulOpposite.lean 2 6 ['github-actions', 'j-loreaux', 'mathlib4-dependent-issues-bot', 'themathqueen'] nobody
7-18798
7 days ago
9-36206
9 days ago
26-57717
26 days
27378 peakpoint
author:peakpoint
refactor(Geometry/Euclidean/Projection): redefine projection and reflection for affine subspaces This PR continues the work from #25578. Original PR: https://github.com/leanprover-community/mathlib4/pull/25578 new-contributor t-euclidean-geometry 316/317 Mathlib/Analysis/Normed/Affine/ContinuousAffineMap.lean,Mathlib/Analysis/Normed/Affine/Isometry.lean,Mathlib/Geometry/Euclidean/Circumcenter.lean,Mathlib/Geometry/Euclidean/Projection.lean 4 4 ['github-actions', 'leanprover-community-bot-assistant', 'peakpoint'] nobody
4-77832
4 days ago
4-78935
4 days ago
8-48270
8 days
24804 Moises-Herradon-Cueto
author:Moises-Herradon-Cueto
feat(CategoryTheory/Limits/Preserves/Shapes): show that if a functor preserves limits, so does `Over.post` If a functor `F` preserves limits (of a certain shape, finite, or of a certain size), then so does the induced functor on `Over` categories. From Toric Co-authored-by: Yaël Dillies --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) toric new-contributor t-category-theory 125/0 Mathlib.lean,Mathlib/CategoryTheory/Limits/Preserves/Shapes/Over.lean,Mathlib/CategoryTheory/WithTerminal/Basic.lean 3 17 ['Moises-Herradon-Cueto', 'YaelDillies', 'erdOne', 'github-actions', 'joelriou'] nobody
4-48809
4 days ago
66-24489
2 months ago
72-28882
72 days
26660 strihanje01
author:strihanje01
feat(Combinatorics/Additive/VerySmallDoubling): weak non-commutative Kneser's theorem add theorem about the structure of a doubling smaller than the golden ratio --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import new-contributor t-combinatorics 859/5 Mathlib/Combinatorics/Additive/VerySmallDoubling.lean 1 61 ['YaelDillies', 'github-actions', 'strihanje01'] nobody
4-20772
4 days ago
21-9844
21 days ago
26-60063
26 days
26099 grunweg
author:grunweg
feat: add IsEmbedding.sumElim_of_separatingNhds Characterise when the Sum.elim of two inducing maps resp. embeddings is an embedding, and deduce that the ranges of the two maps lying in separated neighbourhoods suffices. This is used in my bordism theory project. Co-authored by: @plp127 --- This PR was manually re-created (and migrated to a fork at the same time) from #22137, since that seemed easiest. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-topology 103/0 Mathlib/Data/Sum/Basic.lean,Mathlib/Topology/Constructions/SumProd.lean 2 6 ['ADedecker', 'github-actions', 'grunweg'] nobody
3-34299
3 days ago
44-25473
1 month ago
44-25464
44 days
27008 oliver-butterley
author:oliver-butterley
feat(Dynamics): add `comp_iterate_integrable` If an observable is integrable then the observable formed by composing with iterates of a measure preserving map is also integrable. Co-authored-by: Lua Viana Reis me@lua.blog.br --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-dynamics 34/0 Mathlib.lean,Mathlib/Dynamics/MeasurePreserving/Lemmas.lean 2 1 ['github-actions'] nobody
3-31958
3 days ago
3-32022
3 days ago
21-15322
21 days
27320 Jlh18
author:Jlh18
doc (CategoryTheory/Bicategory/Grothendieck): rename Grothendieck to coGrothendieck Rename `CategoryTheory.Pseudofunctor.Grothendieck` to `CategoryTheory.Pseudofunctor.coGrothendieck`. Currently there are two inconsistent conventions taken in [`CategoryTheory.Grothendieck`](https://leanprover-community.github.io/mathlib4_docs/Mathlib/CategoryTheory/Grothendieck.html#CategoryTheory.Grothendieck) and [`CategoryTheory.Pseudofunctor.Grothendieck`](https://leanprover-community.github.io/mathlib4_docs/Mathlib/CategoryTheory/Bicategory/Grothendieck.html#CategoryTheory.Pseudofunctor.Grothendieck), namely the latter includes an `op` on the indexing category / base category of the Grothendieck construction. Later on, I will make more PRs to introduce the version of `CategoryTheory.Pseudofunctor.Grothendieck` that does not have an `op`. Zulip discussion: [#mathlib4 > Refactor Grothendieck from Pseudofunctor.Grothendieck](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Refactor.20Grothendieck.20from.20Pseudofunctor.2EGrothendieck/with/529165679). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-category-theory 46/38 Mathlib/CategoryTheory/Bicategory/Grothendieck.lean,Mathlib/CategoryTheory/FiberedCategory/Grothendieck.lean 2 5 ['Jlh18', 'github-actions', 'joelriou', 'kckennylau'] nobody
3-28527
3 days ago
3-28677
3 days ago
9-43719
9 days
26842 oliver-butterley
author:oliver-butterley
feat(Mathlib/Dynamics/BirkhoffSum/Average): add lemma `birkhoffAverage_of_invariant` If a function `g` is invariant under a function `f` (i.e., `g ∘ f = g`), then the Birkhoff average of `g` over `f` for `n` iterations is equal to `g`. Requires that `0 < n`. Co-authored-by: Lua Viana Reis - [x] depends on: #26810 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor easy 10/0 Mathlib/Dynamics/BirkhoffSum/Average.lean 1 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
3-26130
3 days ago
3-26153
3 days ago
3-27040
3 days
27006 zhikaip
author:zhikaip
refactor: crossProduct notation Replace `×₃` with `⨯` (`\X` or `\crossproduct`), and manually deprecate the old syntax. See [#mathlib4 > Notation for crossProduct](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Notation.20for.20crossProduct/with/520119542) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data new-contributor t-meta 37/22 Mathlib/Geometry/Euclidean/Angle/Unoriented/CrossProduct.lean,Mathlib/LinearAlgebra/CrossProduct.lean 2 10 ['eric-wieser', 'github-actions', 'j-loreaux', 'kmill', 'madvorak'] nobody
3-25590
3 days ago
21-7214
21 days ago
21-17239
21 days
26840 oliver-butterley
author:oliver-butterley
feat(Mathlib/Dynamics/BirkhoffSum/Average): add 3 BirkhoffAverage lemmas - `birkhoffAverage_add` - `birkhoffAverage_neg` - `birkhoffAverage_sub` - `birkhoffSum_add'` - `birkhoffSum_neg` - `birkhoffSum_sub` Co-authored-by: Lua Viana Reis --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-dynamics 34/1 Mathlib/Dynamics/BirkhoffSum/Average.lean,Mathlib/Dynamics/BirkhoffSum/Basic.lean 2 5 ['ADedecker', 'estradilua', 'github-actions', 'oliver-butterley'] nobody
2-51969
2 days ago
3-30568
3 days ago
25-49864
25 days
27641 FormulaRabbit81
author:FormulaRabbit81
feat: Proof of relative compactness implies tightness of a set of measures (Easy direction of Prokhorov's theorem). PR proving the easy direction of Prokhorov's theorem. I am not sure about the naming conventions and any comments are appreciated. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import new-contributor t-measure-probability 260/1 Mathlib/Analysis/SpecificLimits/Basic.lean,Mathlib/Data/ENNReal/Operations.lean,Mathlib/MeasureTheory/Measure/ProbabilityMeasure.lean,Mathlib/MeasureTheory/Measure/Tight.lean 4 3 ['FormulaRabbit81', 'github-actions', 'themathqueen'] nobody
2-37629
2 days ago
2-57627
2 days ago
3-22467
3 days
27682 FernandoChu
author:FernandoChu
Chore: Added `vecAppend_empty` lemma Added the `vecAppend_empty`. t-data new-contributor 5/0 Mathlib/Data/Fin/VecNotation.lean 1 1 ['github-actions'] nobody
2-27668
2 days ago
2-27668
2 days ago
2-27878
2 days
26945 gasparattila
author:gasparattila
feat(LinearAlgebra/AffineSpace/AffineSubspace): basic properties of `sInf` and `iInf` These properties are analogous to the existing ones for the binary infimum. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra
label:t-algebra$
48/1 Mathlib/LinearAlgebra/AffineSpace/AffineSubspace/Defs.lean 1 4 ['Ruben-VandeVelde', 'gasparattila', 'github-actions'] eric-wieser
assignee:eric-wieser
2-7081
2 days ago
23-11482
23 days ago
23-11528
23 days
26986 WangYiran01
author:WangYiran01
feat(Partition): add bijection for partitions with max part ≤ r ## Summary This PR adds a new theorem `partition_max_equals_bound` to `Mathlib.Combinatorics.Enumerative.Partition`. It constructs a bijection between: - The set of partitions of `n` in which `r ∈ π.parts` and all parts are `≤ r`, and - The set of partitions of `n - r` whose largest part is at most `r`. This provides a constructive proof via removing/adding `r` from/to the partition multiset, in line with classical enumerative combinatorics. ## Implementation notes - The proof uses `Multiset.erase` and `Multiset.cons` with basic properties of `sum`, `sup`, and `Partition` structures. - The bijection is implemented explicitly via `f` and `g`, and proven mutually inverse via `Subtype.ext`. ## Linting - [x] Passes `lake build` - [x] Linter clean (no commandStart or longLine issues) ## Author Contributed by Yiran Wang. new-contributor t-combinatorics 85/0 Mathlib/Combinatorics/Enumerative/Partition.lean 1 2 ['WangYiran01', 'github-actions'] b-mehta
assignee:b-mehta
2-7080
2 days ago
21-44283
21 days ago
21-44327
21 days
26295 DavidJWebb
author:DavidJWebb
feat: filtering lists and bounded quantifiers are primitive recursive A few useful lemmas not explicitly in Primrec.lean : - Filtering for elements from a list that meet a primrec criterion is primrec - Checking whether a list has some element meeting a primrec criterion is primrec - Checking whether every element of a list meets a primrec criterion is primrec - Primitive recursive functions are closed under bounded existential and universal quantifiers --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-computability new-contributor 174/0 Mathlib.lean,Mathlib/Computability/PrimrecFilter.lean 2 65 ['DavidJWebb', 'github-actions', 'grunweg'] nobody
1-84072
1 day ago
1-84268
1 day ago
30-11783
30 days
27705 yonggyuchoimath
author:yonggyuchoimath
feat(RingTheory.Ideal.Height): add trivial cases feat: add trivial cases of Ideal.Height --- This PR updates `RingTheory.Ideal.Height`, which adds two lemmas `Ideal.height_of_subsingleton` and `Ideal.height_bot_eq_zero`. These compute the height of (any) ideal in a zero commutative ring, and the height of the zero ideal in a nonzero commutative ring. new-contributor t-algebra
label:t-algebra$
9/0 Mathlib/RingTheory/Ideal/Height.lean 1 5 ['erdOne', 'github-actions', 'yonggyuchoimath'] nobody
1-71642
1 day ago
1-83096
1 day ago
1-83140
1 day
26453 jburroni
author:jburroni
feat(Data/PNat/Basic): add order-related instances to PNat Add `SuccAddOrder ℕ+` and `NoMaxOrder ℕ+` instances. This allows, for example, the use of lemmas related to `Intervals` built with ℕ+. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-data new-contributor 18/0 Mathlib/Data/PNat/Basic.lean 1 3 ['eric-wieser', 'github-actions', 'jburroni'] ericrbg
assignee:ericrbg
1-39046
1 day ago
36-10867
1 month ago
36-10911
36 days
26790 FlAmmmmING
author:FlAmmmmING
feat(Combinatorics/Enumerative/Bell.lean): define standard Bell number --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-combinatorics 38/1 Mathlib/Combinatorics/Enumerative/Bell.lean 1 11 ['AntoineChambert-Loir', 'FlAmmmmING', 'eric-wieser', 'github-actions', 'kckennylau', 'madvorak'] awainverse
assignee:awainverse
1-39044
1 day ago
27-19723
27 days ago
27-19768
27 days
26793 FlAmmmmING
author:FlAmmmmING
feat(Algebra/Group /ForwardDiff.lean): add five theorems for forward difference --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import new-contributor t-algebra
label:t-algebra$
212/3 Mathlib/Algebra/Group/ForwardDiff.lean 1 35 ['AntoineChambert-Loir', 'DAE123456', 'FlAmmmmING', 'Ruben-VandeVelde', 'github-actions', 'kckennylau', 'madvorak'] mariainesdff
assignee:mariainesdff
1-39043
1 day ago
14-65633
14 days ago
27-18119
27 days
27741 ShreckYe
author:ShreckYe
feat(Algebra/ModEq): add the `IsTrans` instance for `AddCommGroup.ModEq` The `trans` theorem is present for `AddCommGroup.ModEq` but there is no type class instance, while a similar instance is present for `Int.ModEq`, so I guess it should be missing. new-contributor t-algebra easy
label:t-algebra$
3/0 Mathlib/Algebra/ModEq.lean 1 2 ['ShreckYe', 'github-actions'] nobody
1-38877
1 day ago
1-38878
1 day ago
1-39251
1 day
27090 TerenceGitH
author:TerenceGitH
feat(Topology, Archive/Examples): Kuratowski's closure-complement theorem (incl. sharpness) This is the outcome of a course project at Heidelberg University: https://matematiflo.github.io/CompAssistedMath2025/ feat(Topology): Kuratowski's closure-complement theorem "Topology/Kuratowski.lean" proves Kuratowski's closure-complement theorem, which says that if one repeatedly applies the closure and complement operators to a set in a topological space, at most 14 distinct sets can be obtained. feat(Archive/Examples): sharpness of Kuratowski's closure-complement theorem: "Examples/Kuratowski.lean" gives an example of a so-called "14-set" in ℝ, from which exactly 14 distinct sets can be obtained. Co-authored-by: Luis Sand @luiis-sd Co-authored-by: Leon Müller @leondieprobifi Co-authored-by: Junyan Xu @alreadydone --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-topology 386/0 Archive.lean,Archive/Examples/Kuratowski.lean,Mathlib.lean,Mathlib/Topology/Kuratowski.lean 4 8 ['alreadydone', 'github-actions', 'grunweg', 'wwylele'] j-loreaux
assignee:j-loreaux
1-33259
1 day ago
19-6087
19 days ago
19-7429
19 days
27552 Equilibris
author:Equilibris
chore: make typevec.arrow work over different universes This will be needed to allow `M.corec` to be generic across universes --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data new-contributor 16/10 Mathlib/Data/TypeVec.lean 1 3 ['Equilibris', 'github-actions', 'plp127'] nobody
1-32546
1 day ago
5-20357
5 days ago
5-20401
5 days
27511 Nebula691
author:Nebula691
feat(Algebra/QuadraticAlgebra) : Define Quadratic Algebra co-authored-by : Edison Xie co-authored-by : Kenny Lau --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra
label:t-algebra$
418/0 Mathlib.lean,Mathlib/Algebra/QuadraticAlgebra.lean 2 59 ['Whysoserioushah', 'eric-wieser', 'github-actions', 'kckennylau'] nobody
1-5484
1 day ago
6-22221
6 days ago
6-22265
6 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/) new-contributor t-combinatorics 16/0 Mathlib/Combinatorics/SimpleGraph/Trails.lean 1 3 ['IvanRenison', 'github-actions'] kmill
assignee:kmill
1-2140
1 day ago
66-80091
2 months ago
66-80144
66 days
26909 gasparattila
author:gasparattila
feat(LinearAlgebra/Projectivization/Subspace): correspondence between linear and projective subspaces --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra
label:t-algebra$
51/3 Mathlib/LinearAlgebra/Projectivization/Subspace.lean 1 1 ['github-actions'] Vierkantor
assignee:Vierkantor
1-2130
1 day ago
24-5522
24 days ago
24-5570
24 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/) new-contributor t-analysis 365/0 Mathlib.lean,Mathlib/Analysis/Calculus/FDeriv/Partial.lean,Mathlib/Analysis/Normed/Operator/BoundedLinearMaps.lean 3 7 ['YaelDillies', 'agjftucker', 'github-actions', 'igorkhavkine', 'mathlib4-dependent-issues-bot'] sgouezel
assignee:sgouezel
0-83967
23 hours ago
36-48730
1 month ago
37-34467
37 days
27622 ShreckYe
author:ShreckYe
feat(Analysis/SpecialFunctions/Trigonometric): add the missing `tan_sub` and `tan_sub'` functions for both real and complex numbers While working on some proofs, I found that the `tan_sub` theorems are missing, while there are the corresponding`sin_sub` and `cos_sub` theorems. So I'd like to propose adding these for `tan`. new-contributor t-analysis 38/0 Mathlib/Analysis/SpecialFunctions/Trigonometric/Arctan.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Complex.lean 2 4 ['Ruben-VandeVelde', 'ShreckYe', 'github-actions', 'leanprover-community-bot-assistant'] nobody
0-65897
18 hours ago
0-65914
18 hours ago
3-15703
3 days
27577 bjornsolheim
author:bjornsolheim
feat(Data/Fin/Tuple): lemmas on appending finite sequences Prove simple results regarding appending and de-appending of finite sequences. Used to define conical combinations and the conical hull (subsequent PR). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data new-contributor 42/0 Mathlib/Data/Fin/Tuple/Basic.lean 1 19 ['YaelDillies', 'bjornsolheim', 'eric-wieser', 'github-actions'] nobody
0-55943
15 hours ago
0-55943
15 hours ago
2-14927
2 days
26765 KiringYJ
author:KiringYJ
feat(MeasureTheory/PiSystem): add π-λ theorem and SetLike instance Add two small features to `MeasureTheory/PiSystem`: 1. SetLike instance `instance : SetLike (DynkinSystem α) (Set α)` This lets us write `s ⊆ d` and `t ∈ d` for a DynkinSystem `d`, matching usual mathlib style. 2. `DynkinSystem.pi_lambda` lemma Classical π‑λ theorem: if a π‑system `s` is contained in a Dynkin system `d`, every set measurable for `σ(s)` is also in `d`. Currently, mathlib exposes this result only indirectly (e.g. via `generateFrom_eq`). Although logically equivalent, it is not obvious at first glance that those lemmas are the π‑λ theorem. The new lemma states the result in its familiar textbook form, so users can recognise and cite it immediately. Both pieces are under 10 lines, term‑mode only, and do not modify existing APIs. No breaking changes. No dependencies. new-contributor t-measure-probability 13/0 Mathlib/MeasureTheory/PiSystem.lean 1 13 ['EtienneC30', 'KiringYJ', 'github-actions', 'ocfnash'] nobody
0-38111
10 hours ago
1-23958
1 day ago
28-11801
28 days
27816 BGuillemet
author:BGuillemet
feat(CategoryTheory/Sites/SheafOfTypes): composition of a sheaf with uliftFunctor is still a sheaf Prove that if a presheaf of types is a sheaf, then its composition with `uliftFunctor` is still a sheaf. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-category-theory 4/0 Mathlib/CategoryTheory/Sites/SheafOfTypes.lean 1 1 ['github-actions'] nobody
0-33454
9 hours ago
0-33490
9 hours ago
0-33512
9 hours
27819 BGuillemet
author:BGuillemet
feat(CategoryTheory/Yoneda): add curried version of Yoneda lemma for heterogeneous universes, and other version of homNatIso Prove a curried version of `yonedaCompUliftFunctorEquiv`, ie a completely functorial version of the Yoneda lemma with heterogeneous universes. Dually, prove a curried version of `coyonedaCompUliftFunctorEquiv`, ie a completely functorial version of the coYoneda lemma with heterogeneous universes. In addition, prove a functorial version of `FullyFaithful.natEquiv` using `coyoneda` instead of `yoneda` (previously, the only functorial version of `FullyFaithful.natEquiv` were `homNatIso`, which is written using `yoneda`). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-category-theory 162/36 Mathlib/CategoryTheory/Yoneda.lean 1 1 ['github-actions'] nobody
0-32324
8 hours ago
0-32402
8 hours ago
0-32402
9 hours
27815 BGuillemet
author:BGuillemet
feat(CategoryTheory/Limits/Shapes/Products): add limMapPi and sigmaMapColim Add the canonical morphism from a limit to the product over its objects. Prove that it is a monomorphism. Dually, add the canonical morphism to a colimit from the coproduc of its objects and prove that it is an epimorphism. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-category-theory 44/0 Mathlib/CategoryTheory/Limits/Shapes/Products.lean 1 1 ['github-actions'] nobody
0-32090
8 hours ago
0-34018
9 hours ago
0-34043
9 hours
27284 FernandoChu
author:FernandoChu
Chore(CategoryTheory/MorphismProperty/MonoFactorization): Factor out mono factorizations Factored out `MonoFactorisations` from the `Images` file; also rename it to `MonoFactori*z*ations` so it's inline with the rest of Mathlib. I'm also sneaking in some very basic extremal epis results if you don't mind, these were meant to be used to prove ```lean instance (priority := 100) hasStrongEpiImages_of_hasPullbacks_of_hasEqualizers [HasPullbacks C] [HasEqualizers C] : HasStrongEpiImages C ``` Which I noticed too late already had a proof; I think the proof has been improved anyways, it's just `infer_instance` now. new-contributor t-category-theory 468/312 Mathlib.lean,Mathlib/Algebra/Category/Grp/Images.lean,Mathlib/Algebra/Category/ModuleCat/Images.lean,Mathlib/AlgebraicTopology/SimplexCategory/Basic.lean,Mathlib/CategoryTheory/Abelian/Basic.lean,Mathlib/CategoryTheory/Category/Factorisation.lean,Mathlib/CategoryTheory/ConcreteCategory/EpiMono.lean,Mathlib/CategoryTheory/Limits/Preserves/Shapes/Images.lean,Mathlib/CategoryTheory/Limits/Shapes/ExtremalEpi.lean,Mathlib/CategoryTheory/Limits/Shapes/Images.lean,Mathlib/CategoryTheory/Limits/Shapes/Kernels.lean,Mathlib/CategoryTheory/Limits/Shapes/StrongEpi.lean,Mathlib/CategoryTheory/Limits/Shapes/ZeroMorphisms.lean,Mathlib/CategoryTheory/Limits/Types/Images.lean,Mathlib/CategoryTheory/MorphismProperty/MonoFactorization.lean,Mathlib/CategoryTheory/Sites/Subsheaf.lean,Mathlib/Order/Category/NonemptyFinLinOrd.lean,scripts/nolints_prime_decls.txt 18 29 ['FernandoChu', 'github-actions', 'joelriou', 'robin-carlier'] TwoFX
assignee:TwoFX
0-28302
7 hours ago
0-28392
7 hours ago
13-31623
13 days
27825 yonggyuchoimath
author:yonggyuchoimath
feat(RingTheory/Ideal/Height): sup of ideal heights equals Krull dimension feat: sup of ideal heights equals Krull dimension --- This PR adds `Ideal.sup_height_eq_ringKrullDim` `Ideal.sup_primeHeight_eq_ringKrullDim` They show the suprema of heights of ideals / prime ideals are equal to the Krull dimension, when the ring is nonzero. new-contributor t-algebra
label:t-algebra$
53/0 Mathlib/RingTheory/Ideal/Height.lean 1 2 ['github-actions', 'yonggyuchoimath'] nobody
0-27921
7 hours ago
0-29520
8 hours ago
0-29568
8 hours
27755 bwangpj
author:bwangpj
feat(RepresentationTheory/Basic): direct sum of representations Define the `DirectSum` of a family of `Representation`s. [Zulip thread](https://leanprover.zulipchat.com/#narrow/channel/116395-maths/topic/Representation.20Theory) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra
label:t-algebra$
39/0 Mathlib/RepresentationTheory/Basic.lean 1 3 ['bwangpj', 'github-actions', 'kbuzzard'] nobody
0-27390
7 hours ago
1-22233
1 day ago
1-22279
1 day
26272 ajirving
author:ajirving
feat(NumberTheory/LucasLehmer): prove converse direction to Lucas-Lehmer Proves the converse direction of the Lucas-Lehmer test, namely that the Lucas-Lehmer criterion is a necessary condition for a Mersenne prime. Adds a couple of examples of proving Mersenne numbers are composite using this. Proves that if `2^p-1` is prime then `p` is prime. --- * I wasn't sure how many examples to add given that there are many more Mersenne composites than primes. * There are a number of annoying coercions between different rings, any simplifications will be appreciated. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import new-contributor t-number-theory 226/5 Archive/Examples/MersennePrimes.lean,Mathlib/NumberTheory/LucasLehmer.lean 2 12 ['github-actions', 'kckennylau'] kbuzzard
assignee:kbuzzard
0-17613
4 hours ago
40-22302
1 month ago
40-22347
40 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/) new-contributor t-algebra
label:t-algebra$
106/0 Mathlib/GroupTheory/DoubleCoset.lean 1 1 ['github-actions'] mariainesdff
assignee:mariainesdff
0-17607
4 hours ago
15-21359
15 days ago
15-21409
15 days
27400 dleijnse
author:dleijnse
feat: define geometrically reduced algebras Define geometrically reduced algebras, and prove that if all finitely generated subalgebras of an algebra `A` are geometrically reduced, then `A` is geometrically reduced. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra
label:t-algebra$
111/0 Mathlib.lean,Mathlib/RingTheory/Nilpotent/GeometricallyReduced.lean 2 23 ['dleijnse', 'github-actions', 'kckennylau'] nobody
0-14497
4 hours ago
9-6574
9 days ago
9-6619
9 days
27663 ShreckYe
author:ShreckYe
feat(Analysis/SpecialFunctions/Trigonometric/Basic): add the duals named `cos_eq_zero_iff_sin_eq` for the theorems named `sin_eq_zero_iff_cos_eq` in both real and complex cases Similar to #27622. These seem missing for cosine case. I simplified the proofs adapted from `sin_eq_zero_iff_cos_eq` using `simp` compared to the original way of constructing the remaining goal explictly using `exact`. If needed, I can simplify the proofs of the 2 `sin_eq_zero_iff_cos_eq`s too. new-contributor t-analysis easy 8/0 Mathlib/Analysis/SpecialFunctions/Trigonometric/Basic.lean 1 6 ['ShreckYe', 'github-actions', 'themathqueen'] nobody
0-9927
2 hours ago
1-38671
1 day ago
2-69922
2 days
24527 matthewjasper
author:matthewjasper
feat(Topology/Algebra/Module): Add more theorems for IsModuleTopology Add theorems that surjective linear maps to the module topology are open. Add IsModuleTopology instance for quotients. Add IsModuleTopology instance for finite dimensional T2 vector spaces over a complete normed field and use it to shorten some proofs. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra t-topology
label:t-algebra$
52/26 Mathlib/Analysis/Fourier/AddCircleMulti.lean,Mathlib/Analysis/RCLike/Lemmas.lean,Mathlib/Topology/Algebra/Module/FiniteDimension.lean,Mathlib/Topology/Algebra/Module/ModuleTopology.lean 4 8 ['erdOne', 'github-actions', 'matthewjasper', 'ocfnash', 'riccardobrasca'] ocfnash
assignee:ocfnash
0-387
6 minutes ago
90-35968
2 months ago
92-4263
92 days

PRs on the review queue labelled 'easy'

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
27110 pechersky
author:pechersky
chore(Valued/WithVal): apply_symm_equiv valuation on the WIthVal is equal to the underlying valuation and simp tag --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-topology t-number-theory easy
label:t-algebra$
4/0 Mathlib/Topology/Algebra/Valued/WithVal.lean 1 1 ['github-actions'] nobody
18-62952
18 days ago
18-62955
18 days ago
18-63009
18 days
26842 oliver-butterley
author:oliver-butterley
feat(Mathlib/Dynamics/BirkhoffSum/Average): add lemma `birkhoffAverage_of_invariant` If a function `g` is invariant under a function `f` (i.e., `g ∘ f = g`), then the Birkhoff average of `g` over `f` for `n` iterations is equal to `g`. Requires that `0 < n`. Co-authored-by: Lua Viana Reis - [x] depends on: #26810 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor easy 10/0 Mathlib/Dynamics/BirkhoffSum/Average.lean 1 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
3-26130
3 days ago
3-26153
3 days ago
3-27040
3 days
27634 agjftucker
author:agjftucker
fix(Analysis/Calculus/Implicit): consistently rename {`map`, `fun`, `function`} to `fun` There are several clear naming issues in the file Implicit.lean, such as ``` theorem prod_map_implicitFunction : ∀ᶠ p : F × G in 𝓝 (φ.prodFun φ.pt), φ.prodFun (φ.implicitFunction p.1 p.2) = p := ``` where `prod_map` and `prodFun` both refer to the same thing. In this PR I have done my best to resolve these as consistently as possible by renaming everything `map`, also everything `function`, to `fun`. This has the added benefit of making some long names a little shorter. In passing I rewrapped some comments and replaced `haveI` with `have` where it had been used like `haveI` in Lean 3. Moves: - ImplicitFunctionData -> ImplicitFunData - ImplicitFunctionData.implicitFunction -> ImplicitFunData.implicitFun - ImplicitFunctionData.prod_map_implicitFunction -> ImplicitFunData.prodFun_implicitFun - ImplicitFunctionData.left_map_implicitFunction -> ImplicitFunData.leftFun_implicitFun - ImplicitFunctionData.right_map_implicitFunction -> ImplicitFunData.rightFun_implicitFun - ImplicitFunctionData.implicitFunction_apply_image -> ImplicitFunData.implicitFun_apply_image - ImplicitFunctionData.implicitFunction_hasStrictFDerivAt -> ImplicitFunData.hasStrictFDerivAt_implicitFun - HasStrictFDerivAt.implicitFunctionDataOfComplemented -> HasStrictFDerivAt.implicitFunDataOfComplemented - HasStrictFDerivAt.implicitFunctionOfComplemented -> HasStrictFDerivAt.implicitFunOfComplemented - HasStrictFDerivAt.map_implicitFunctionOfComplemented_eq -> HasStrictFDerivAt.map_implicitFunOfComplemented_eq - HasStrictFDerivAt.eq_implicitFunctionOfComplemented -> HasStrictFDerivAt.eq_implicitFunOfComplemented - HasStrictFDerivAt.implicitFunctionOfComplemented_apply_image -> HasStrictFDerivAt.implicitFunOfComplemented_apply_image - HasStrictFDerivAt.to_implicitFunctionOfComplemented -> HasStrictFDerivAt.to_implicitFunOfComplemented - HasStrictFDerivAt.implicitFunction -> HasStrictFDerivAt.implicitFun - HasStrictFDerivAt.tendsto_implicitFunction -> HasStrictFDerivAt.tendsto_implicitFun - _root_.Filter.Tendsto.implicitFunction -> _root_.Filter.Tendsto.implicitFun - HasStrictFDerivAt.map_implicitFunction_eq -> HasStrictFDerivAt.map_implicitFun_eq - HasStrictFDerivAt.implicitFunction_apply_image -> HasStrictFDerivAt.implicitFun_apply_image - HasStrictFDerivAt.eq_implicitFunction -> HasStrictFDerivAt.eq_implicitFun - HasStrictFDerivAt.to_implicitFunction -> HasStrictFDerivAt.to_implicitFun --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis easy 165/121 Mathlib/Analysis/Calculus/Implicit.lean,docs/1000.yaml,docs/overview.yaml,docs/undergrad.yaml 4 1 ['github-actions'] nobody
3-13432
3 days ago
3-34878
3 days ago
3-34926
3 days
27665 pechersky
author:pechersky
chore(Algebra/Group/WithOne): With{One,Zero}.coe_injective --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra easy
label:t-algebra$
4/0 Mathlib/Algebra/Group/WithOne/Defs.lean 1 1 ['github-actions'] nobody
2-60360
2 days ago
2-60534
2 days ago
2-60530
2 days
27549 Ruben-VandeVelde
author:Ruben-VandeVelde
feat: Submodule.smul_one_eq_span Co-authored-by: Aaron Hill Co-authored-by: Austin Letson Co-authored-by: Matej Penciak --- From FLT [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) FLT t-algebra easy
label:t-algebra$
3/0 Mathlib/Algebra/Algebra/Operations.lean 1 3 ['github-actions', 'ocfnash'] nobody
2-23812
2 days ago
5-22916
5 days ago
5-22963
5 days
27685 ocfnash
author:ocfnash
feat: add `Pi.evalLinear` (evaluation as a linear map) --- I'm amazed this seems not to exist already but I can't find it after looking carefully. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-algebra easy
label:t-algebra$
24/1 Mathlib/Algebra/Module/Pi.lean,Mathlib/Order/Filter/Germ/Basic.lean 2 1 ['github-actions'] nobody
2-23172
2 days ago
2-24507
2 days ago
2-25287
2 days
27703 vihdzp
author:vihdzp
feat: `le_of_forall_ne` This form of `le_of_forall_lt` is a bit nicer when working with nimbers; they're minimum excludents, so to prove `a ≤ b` you have to prove `b` can't be equal to any smaller `a`! --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order easy 7/0 Mathlib/Order/Basic.lean 1 1 ['github-actions'] nobody
1-76452
1 day ago
1-85686
1 day ago
1-85687
1 day
27741 ShreckYe
author:ShreckYe
feat(Algebra/ModEq): add the `IsTrans` instance for `AddCommGroup.ModEq` The `trans` theorem is present for `AddCommGroup.ModEq` but there is no type class instance, while a similar instance is present for `Int.ModEq`, so I guess it should be missing. new-contributor t-algebra easy
label:t-algebra$
3/0 Mathlib/Algebra/ModEq.lean 1 2 ['ShreckYe', 'github-actions'] nobody
1-38877
1 day ago
1-38878
1 day ago
1-39251
1 day
27794 xroblot
author:xroblot
feat(RingTheory): add `symm_apply_eq` and `eq_symm_apply` for `RingEquiv` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra easy
label:t-algebra$
6/0 Mathlib/Algebra/Ring/Equiv.lean 1 1 ['github-actions'] nobody
0-69967
19 hours ago
0-69980
19 hours ago
0-70024
19 hours
27807 grunweg
author:grunweg
chore: mark Polynomial.differential fun_prop And remove a superfluous `local fun_prop` tag: Complex.continuous_abs is already marked fun_prop. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) easy 1/3 Mathlib/Analysis/Calculus/Deriv/Polynomial.lean,Mathlib/NumberTheory/Transcendental/Lindemann/AnalyticalPart.lean 2 1 ['github-actions'] nobody
0-42963
11 hours ago
0-43030
11 hours ago
0-43014
11 hours
27822 Louddy
author:Louddy
feat(RatFunc): theorems algebraMap polynomial Two simple lemmas about the `algebraMap` from `F[X]` to `RatFunc F`: - A `monomial n a` is `C a * X ^ n` (here we are using `RatFunc.X` and `RatFunc.C`.) - The algebraMap from `F[X]` to `RatFunc F` is the same as the evaluation of a polynomial `p` at `RatFunc.X`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra easy
label:t-algebra$
9/0 Mathlib/FieldTheory/RatFunc/AsPolynomial.lean 1 1 ['github-actions'] nobody
0-30293
8 hours ago
0-30293
8 hours ago
0-30443
8 hours
27035 faenuccio
author:faenuccio
chore(IsManifold/Basic): replace continuity by aesop --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-differential-geometry easy 5/5 Mathlib/Geometry/Manifold/IsManifold/Basic.lean 1 3 ['faenuccio', 'fpvandoorn', 'github-actions'] sgouezel
assignee:sgouezel
0-17609
4 hours ago
20-18703
20 days ago
20-21590
20 days
27248 kckennylau
author:kckennylau
chore: remove `suppress_compilation` from Mathlib.Algebra.Category.Ring.Constructions --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra easy
label:t-algebra$
2/4 Mathlib/Algebra/Category/Ring/Constructions.lean 1 4 ['github-actions', 'grunweg', 'leanprover-bot'] chrisflav
assignee:chrisflav
0-17606
4 hours ago
14-36412
14 days ago
14-36460
14 days
27663 ShreckYe
author:ShreckYe
feat(Analysis/SpecialFunctions/Trigonometric/Basic): add the duals named `cos_eq_zero_iff_sin_eq` for the theorems named `sin_eq_zero_iff_cos_eq` in both real and complex cases Similar to #27622. These seem missing for cosine case. I simplified the proofs adapted from `sin_eq_zero_iff_cos_eq` using `simp` compared to the original way of constructing the remaining goal explictly using `exact`. If needed, I can simplify the proofs of the 2 `sin_eq_zero_iff_cos_eq`s too. new-contributor t-analysis easy 8/0 Mathlib/Analysis/SpecialFunctions/Trigonometric/Basic.lean 1 6 ['ShreckYe', 'github-actions', 'themathqueen'] nobody
0-9927
2 hours ago
1-38671
1 day ago
2-69922
2 days

PRs on the review queue labelled 'tech debt' or 'longest-pole'

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
25776 Parcly-Taxel
author:Parcly-Taxel
chore: deprime `induction` in `Analysis` I think this is very marginally dependent on #25770. tech debt t-analysis 256/208 Mathlib/Analysis/Analytic/Composition.lean,Mathlib/Analysis/Analytic/Constructions.lean,Mathlib/Analysis/Analytic/Inverse.lean,Mathlib/Analysis/BoxIntegral/Basic.lean,Mathlib/Analysis/BoxIntegral/Box/SubboxInduction.lean,Mathlib/Analysis/BoxIntegral/Partition/Additive.lean,Mathlib/Analysis/BoxIntegral/Partition/Split.lean,Mathlib/Analysis/CStarAlgebra/Basic.lean,Mathlib/Analysis/CStarAlgebra/Multiplier.lean,Mathlib/Analysis/Calculus/ContDiff/Basic.lean,Mathlib/Analysis/Calculus/ContDiff/Bounds.lean,Mathlib/Analysis/Calculus/ContDiff/FTaylorSeries.lean,Mathlib/Analysis/Calculus/ContDiff/Operations.lean,Mathlib/Analysis/Calculus/Deriv/ZPow.lean,Mathlib/Analysis/Calculus/InverseFunctionTheorem/ApproximatesLinearOn.lean,Mathlib/Analysis/Calculus/IteratedDeriv/Lemmas.lean,Mathlib/Analysis/Calculus/SmoothSeries.lean,Mathlib/Analysis/Convex/Combination.lean,Mathlib/Analysis/Convex/Radon.lean,Mathlib/Analysis/InnerProductSpace/Projection.lean,Mathlib/Analysis/Normed/Algebra/Exponential.lean,Mathlib/Analysis/NormedSpace/Multilinear/Basic.lean,Mathlib/Analysis/Seminorm.lean,Mathlib/Analysis/SpecialFunctions/Complex/Arg.lean,Mathlib/Analysis/SpecialFunctions/Complex/Circle.lean,Mathlib/Analysis/SpecialFunctions/Gamma/Basic.lean,Mathlib/Analysis/SpecialFunctions/Gamma/Beta.lean,Mathlib/Analysis/SpecialFunctions/Gamma/BohrMollerup.lean,Mathlib/Analysis/SpecialFunctions/Gamma/Deriv.lean,Mathlib/Analysis/SpecialFunctions/Integrals/Basic.lean,Mathlib/Analysis/SpecialFunctions/Log/Basic.lean,Mathlib/Analysis/SpecialFunctions/Pow/Deriv.lean,Mathlib/Analysis/SpecialFunctions/Pow/NNReal.lean,Mathlib/Analysis/SpecialFunctions/Pow/Real.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/EulerSineProd.lean 35 3 ['Parcly-Taxel', 'github-actions', 'leanprover-community-bot-assistant', 'madvorak'] nobody
25-39140
25 days ago
25-73112
25 days ago
48-53287
48 days
25770 Parcly-Taxel
author:Parcly-Taxel
chore: fix more induction/recursor branch names These were found using the regex `\| h. =>` and `def.*rec.*\(h. :`. tech debt 134/115 Mathlib/Analysis/Convolution.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/Data/Fin/Tuple/Basic.lean,Mathlib/Data/Fin/Tuple/NatAntidiagonal.lean,Mathlib/Data/Nat/Factorization/Induction.lean,Mathlib/Data/Seq/Computation.lean,Mathlib/Data/Set/Card.lean,Mathlib/Data/WSeq/Basic.lean,Mathlib/FieldTheory/KummerExtension.lean,Mathlib/Logic/Function/Iterate.lean,Mathlib/NumberTheory/ArithmeticFunction.lean,Mathlib/NumberTheory/SumFourSquares.lean,Mathlib/NumberTheory/SumTwoSquares.lean,Mathlib/Order/SuccPred/Archimedean.lean,Mathlib/Order/Synonym.lean 15 11 ['Parcly-Taxel', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant'] nobody
16-69283
16 days ago
25-73346
25 days ago
48-55733
48 days
27455 pechersky
author:pechersky
chore(NumberTheory/Padics/Hensel): rephrase using `aeval` This is easier to use at call site, because on need not pass `Polynomial.map (algebraMap _ _ )` in the use of `hensels_lemma` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) tech debt t-algebra t-number-theory
label:t-algebra$
157/138 Mathlib/NumberTheory/Padics/Hensel.lean 1 1 ['github-actions'] nobody
7-68304
7 days ago
7-68359
7 days ago
7-68356
7 days
26270 vasnesterov
author:vasnesterov
chore(Analysis/Analytic): split `Analytic.Basic` Move the results on the radius of convergence from `Analytic/Basic.lean` to a new file `Analytic/ConvergenceRadius.lean`. --- - [x] depends on: #26255 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) tech debt t-analysis 450/431 Mathlib.lean,Mathlib/Analysis/Analytic/Basic.lean,Mathlib/Analysis/Analytic/ConvergenceRadius.lean,Mathlib/Analysis/Analytic/OfScalars.lean,Mathlib/Analysis/Analytic/RadiusLiminf.lean 5 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
5-35334
5 days ago
5-35334
5 days ago
6-25073
6 days
25774 Parcly-Taxel
author:Parcly-Taxel
chore: deprime `induction` in `AlgebraicTopology/CategoryTheory` Most replacements that are also in #23676 have been copied over, but some have been optimised further. tech debt 130/121 Mathlib/AlgebraicTopology/DoldKan/Decomposition.lean,Mathlib/AlgebraicTopology/DoldKan/Degeneracies.lean,Mathlib/AlgebraicTopology/DoldKan/NCompGamma.lean,Mathlib/AlgebraicTopology/DoldKan/Projections.lean,Mathlib/AlgebraicTopology/SimplexCategory/MorphismProperty.lean,Mathlib/AlgebraicTopology/SimplicialObject/Split.lean,Mathlib/AlgebraicTopology/SimplicialSet/Degenerate.lean,Mathlib/AlgebraicTopology/SimplicialSet/NerveAdjunction.lean,Mathlib/AlgebraicTopology/SimplicialSet/StdSimplex.lean,Mathlib/CategoryTheory/Abelian/GrothendieckCategory/EnoughInjectives.lean,Mathlib/CategoryTheory/Abelian/GrothendieckCategory/Subobject.lean,Mathlib/CategoryTheory/Action/Concrete.lean,Mathlib/CategoryTheory/Action/Monoidal.lean,Mathlib/CategoryTheory/ComposableArrows.lean,Mathlib/CategoryTheory/Extensive.lean,Mathlib/CategoryTheory/Filtered/Basic.lean,Mathlib/CategoryTheory/Galois/Decomposition.lean,Mathlib/CategoryTheory/Galois/EssSurj.lean,Mathlib/CategoryTheory/Limits/Shapes/Equalizers.lean,Mathlib/CategoryTheory/Limits/Shapes/SequentialProduct.lean,Mathlib/CategoryTheory/Limits/VanKampen.lean,Mathlib/CategoryTheory/Quotient.lean,Mathlib/CategoryTheory/Sites/Sheaf.lean,Mathlib/CategoryTheory/Subobject/Basic.lean,Mathlib/CategoryTheory/Subobject/FactorThru.lean,Mathlib/CategoryTheory/Subobject/Lattice.lean,Mathlib/CategoryTheory/Triangulated/TStructure/Basic.lean 27 6 ['Parcly-Taxel', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'madvorak'] nobody
3-21246
3 days ago
3-21265
3 days ago
48-13756
48 days
27339 pechersky
author:pechersky
chore(RingTheory/Laurent): use WithZero.exp to golf statements and proofs about valuation on K((X)) Done as part of refactor of Valued in #27314. This PR does not change any definitions. Instead, uses `WithZero.exp` instead of coercion + Multiplicative.ofAdd. And some helper simp lemmas about valuations of RatFunc vis a vis LaurentSeries. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) tech debt t-algebra t-number-theory
label:t-algebra$
78/77 Mathlib/FieldTheory/RatFunc/AsPolynomial.lean,Mathlib/RingTheory/LaurentSeries.lean,Mathlib/Topology/Algebra/Valued/WithVal.lean 3 1 ['github-actions'] Vierkantor
assignee:Vierkantor
1-45408
1 day ago
10-24187
10 days ago
10-68182
10 days
27439 Vierkantor
author:Vierkantor
chore(*): review 2024-04-01 adaptation notes There are three kinds of adaptation notes from the changes on 2024-04-01. One about `erw` "blowing up"; this referred to a backwards compatibility flag that was already removed long ago (#14064). So this can just be deleted. A few about needing to use `symm` before `ext` fires: this is because `apply` failing to unify when mixing very general limit definitions and very specific operations for equalizers/pullbacks. I propose we fix this by unfolding the terms manually in an `intro` type ascription. In the longer term we should consider instead specializing the limit lemmas to these specific shapes. A few about `aesop` not working. This has the same underlying cause, due to `ext` not applying, so it now looks like `intro s (m : _ --> _) x; aesop`. Same specializing of the limit lemmas may be useful here. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) tech debt 8/25 Mathlib/AlgebraicGeometry/Spec.lean,Mathlib/CategoryTheory/Limits/Shapes/KernelPair.lean,Mathlib/CategoryTheory/Limits/Shapes/Kernels.lean,Mathlib/CategoryTheory/Limits/Shapes/Products.lean 4 2 ['github-actions', 'grunweg'] jcommelin
assignee:jcommelin
0-40451
11 hours ago
8-13083
8 days ago
8-13066
8 days