Mathlib triage dashboard

Welcome to the PR triage page! This page is perfect if you intend to look for pull request which seem to have stalled.
Feedback on designing this page or further information to include is very welcome.

This dashboard was last updated on: June 09, 2025 at 20:06 UTC

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

Overall statistics

Found 1544 open PRs overall. Among these PRs

Approved, not yet landed PRs

At the moment,

Review status

There are currently 301 PRs awaiting review. Among these,

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

Stale unassigned PRs on the review queue

Number Author Title Description Labels +/- Modified files (first 100) 📝 💬 All users who commented or reviewed Assignee(s) Approval(s) Updated Last status change total time in review
24218 alreadydone
author:alreadydone
chore(Algebra): remove `mid_assoc` from `IsMulCentral` as it is a consequence of left and right associativity in the presence of commutativity. Also change the commutativity condition to use `Commute`. --- Even without commutativity, left and right associativity of an element `e` in a magma is sufficient to prove that elements of the form `e * x * e` (the "corner" of `e`) form a submagma. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
31/69 Mathlib/Algebra/Algebra/NonUnitalSubalgebra.lean,Mathlib/Algebra/Group/Center.lean,Mathlib/Algebra/GroupWithZero/Center.lean,Mathlib/Algebra/Ring/Center.lean,Mathlib/Algebra/Ring/CentroidHom.lean,Mathlib/Algebra/Star/Center.lean,Mathlib/Algebra/Star/CentroidHom.lean,Mathlib/GroupTheory/Submonoid/Center.lean,Mathlib/LinearAlgebra/Basis/Submodule.lean,Mathlib/LinearAlgebra/QuadraticForm/Basic.lean,Mathlib/RingTheory/Idempotents.lean,Mathlib/RingTheory/NonUnitalSubsemiring/Basic.lean 12 8 ['alreadydone', 'github-actions', 'mans0954'] nobody 1
50-12169
1 month ago
50-27229
1 month ago
50-27219
50 days
24394 wwylele
author:wwylele
feat(Analysis/Asymptotics): Add filter operation theorems to `IsEquivalent` These are simply restating the corresponding theorems for `isLittleO`, but adding them provides better discovery when one is not familiar with how `IsEquivalent` is defined. I tagged `isEquivalent_map` as `@[simp]` because all of `isBigOWith/isBigO/isLittleO_map` are tagged, but I am not sure if this appropriate. Please let me know if I should remove the tag --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-analysis 13/0 Mathlib/Analysis/Asymptotics/AsymptoticEquivalent.lean 1 1 ['github-actions'] nobody none
44-3314
1 month ago
44-3314
1 month ago
44-3373
44 days
24405 mcdoll
author:mcdoll
refactor(Topology/Algebra/Module/WeakDual): Clean up - Move `Dual` and `dualPairing` lower in the import-hierachy - deduplicate `dualPairing` - Make `WeakDual` and `WeakSpace` reducible --- New version of #11500 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-topology 146/162 Mathlib.lean,Mathlib/Analysis/Fourier/RiemannLebesgueLemma.lean,Mathlib/Analysis/InnerProductSpace/Adjoint.lean,Mathlib/Analysis/InnerProductSpace/Dual.lean,Mathlib/Analysis/LocallyConvex/WeakSpace.lean,Mathlib/Analysis/Normed/Module/Dual.lean,Mathlib/Analysis/Normed/Module/WeakDual.lean,Mathlib/Analysis/VonNeumannAlgebra/Basic.lean,Mathlib/MeasureTheory/Function/AEEqOfIntegral.lean,Mathlib/MeasureTheory/Measure/FiniteMeasure.lean,Mathlib/Topology/Algebra/Module/Dual.lean,Mathlib/Topology/Algebra/Module/WeakDual.lean,docs/overview.yaml,docs/undergrad.yaml 14 1 ['github-actions'] nobody none
42-65841
1 month ago
42-74534
1 month ago
42-74517
42 days
24266 plp127
author:plp127
feat(Order): `NoBotOrder α` implies `NoMinOrder α` under `IsDirected α (· ≥ ·)` Proves that `NoBotOrder α` implies `NoMinOrder α` under `IsDirected α (· ≥ ·)`, and also the dual theorem. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order 14/0 Mathlib/Order/Directed.lean 1 4 ['github-actions', 'plp127', 'urkud'] nobody none
37-63061
1 month ago
48-74442
1 month ago
48-74426
48 days
23498 Ruben-VandeVelde
author:Ruben-VandeVelde
chore(Topology.MetricSpace.Lipschitz): stop depending on Topology.Algebra Noticed while playing with the new `directoryDependency` linter. Not sure if these could be proved without assuming the continuity of real multiplication. Copyright from https://github.com/leanprover-community/mathlib3/pull/1921 and https://github.com/leanprover-community/mathlib4/pull/11840. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology 60/34 Mathlib.lean,Mathlib/Analysis/Normed/Group/AddTorsor.lean,Mathlib/Analysis/NormedSpace/Multilinear/Basic.lean,Mathlib/Analysis/SpecialFunctions/Exp.lean,Mathlib/Topology/Algebra/MetricSpace/Lipschitz.lean,Mathlib/Topology/MetricSpace/Algebra.lean,Mathlib/Topology/MetricSpace/IsometricSMul.lean,Mathlib/Topology/MetricSpace/Lipschitz.lean,Mathlib/Topology/MetricSpace/PiNat.lean 9 1 ['github-actions'] nobody none
37-46198
1 month ago
37-46198
1 month ago
70-25921
70 days
23360 kim-em
author:kim-em
chore: review of `erw` in `Algebra/Homology/DerivedCategory` t-algebra
label:t-algebra$
21/15 Mathlib/Algebra/Homology/DerivedCategory/Basic.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/ExtClass.lean,Mathlib/Algebra/Homology/DerivedCategory/SingleTriangle.lean,Mathlib/Algebra/Homology/HomotopyCategory/SingleFunctors.lean,Mathlib/CategoryTheory/Shift/SingleFunctors.lean 5 2 ['Ruben-VandeVelde', 'github-actions'] nobody none
37-46186
1 month ago
37-46186
1 month ago
74-57653
74 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$
48/24 Mathlib/Topology/Algebra/Module/FiniteDimension.lean,Mathlib/Topology/Algebra/Module/ModuleTopology.lean 2 5 ['erdOne', 'github-actions', 'matthewjasper'] nobody none
37-13321
1 month ago
37-30391
1 month ago
38-85090
38 days
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 none
36-59820
1 month ago
105-61462
3 months ago
105-61587
105 days
24361 Hagb
author:Hagb
feat(Data/Finsupp/MonomialOrder): `0 ≤ a` where `a : m.syn` `simp` would be able to solve it. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data new-contributor easy 3/0 Mathlib/Data/Finsupp/MonomialOrder.lean 1 1 ['github-actions'] nobody none
33-42488
1 month ago
33-42488
1 month ago
45-44165
45 days
24711 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/) 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 8 ['github-actions', 'joelriou', 'robin-carlier'] nobody none
30-34702
30 days ago
30-34702
30 days ago
31-17992
31 days
24351 eric-wieser
author:eric-wieser
feat: fderiv lemmas for `pow` This generalizes the lemmas about `fderiv fun x => f x ^ n` to work over arbitrary normed modules and algebras. Following the convention set by the lemmas about `fderiv` and `*`, we use `'`d names for the non-commutative variants. Moves: - `deriv_pow''` -> `deriv_pow` - `deriv_pow` -> `deriv_pow_field` - `derivWithin_pow'` -> `derivWithin_pow_field'` Deletions: - `deriv_pow'` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis 282/82 Mathlib.lean,Mathlib/Analysis/Calculus/Deriv/Polynomial.lean,Mathlib/Analysis/Calculus/Deriv/Pow.lean,Mathlib/Analysis/Calculus/FDeriv/Mul.lean,Mathlib/Analysis/Calculus/FDeriv/Pow.lean,Mathlib/Analysis/Calculus/Taylor.lean,Mathlib/Analysis/Complex/Angle.lean,Mathlib/Analysis/Convex/SpecificFunctions/Deriv.lean,Mathlib/NumberTheory/ModularForms/JacobiTheta/TwoVariable.lean 9 2 ['github-actions', 'leanprover-community-bot-assistant'] nobody none
29-68522
29 days ago
29-68522
29 days ago
30-15569
30 days
22966 alreadydone
author:alreadydone
feat(RingTheory): degree of rational function field extension + `IsAlgebraic/IsIntegral R S` + `IsPushout R S R' S'` ⇒ `IsAlgebraic/IsIntegral R' S'` (for the "IsAlgebraic" version we currently need to assume `NoZeroDivisor R'` and `FaithfulSMul R R'` (i.e. `Injective (algebraMap R R')`) + `IsAlgebraic R S` + `IsFractionRing R R'` + `IsFractionRing S S'` ⇒ `IsPushout R S R' S'` (need to assume `FaithfulSMul R S` + `NonZeroDivisors S`) As consequences, we have `rank (f R) (f S) = rank R S` for `f = FractionRing (Polynomial ·)` or `FractionRing (MvPolynomial _ ·)` assuming `IsAlgebraic R S` + `IsDomain S` + `FaithfulSMul R S`. (For `f = Polynomial` or `MvPolynomial _`, `NoZeroDivisors R` is enough by #23095.) --- - [x] depends on: #23095 - [x] depends on: #23096 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
272/49 Mathlib/RingTheory/AdjoinRoot.lean,Mathlib/RingTheory/Algebraic/Basic.lean,Mathlib/RingTheory/Algebraic/Integral.lean,Mathlib/RingTheory/AlgebraicIndependent/AlgebraicClosure.lean,Mathlib/RingTheory/IntegralClosure/IsIntegralClosure/Basic.lean,Mathlib/RingTheory/TensorProduct/Basic.lean 6 11 ['Louddy', 'alreadydone', 'github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody none
29-64005
29 days ago
29-64974
29 days ago
47-35835
47 days
24602 xyzw12345
author:xyzw12345
feat(LinearAlgebra/SymmetricAlgebra): IsSymmetricAlgebra This PR is a part of #21539, which separates out the part about `IsSymmetricAlgebra`. Co-authored-by: Raphael Douglas Giles @Raph-DG Co-authored-by: Zhixuan Dai <22300180006@m.fudan.edu.cn> Co-authored-by: Zhenyan Fu Co-authored-by: Yiming Fu - [ ] depends on: #21539 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
78/0 Mathlib/LinearAlgebra/SymmetricAlgebra/Basic.lean,Mathlib/LinearAlgebra/SymmetricAlgebra/Basis.lean 2 5 ['eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody none
29-11986
29 days ago
29-12238
29 days ago
29-14179
29 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 none
29-1394
29 days ago
29-7345
29 days ago
76-59566
76 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 11 ['eric-wieser', 'github-actions', 'mathlib4-dependent-issues-bot', 'plp127', 'vihdzp'] nobody none
28-72193
28 days ago
28-73125
28 days ago
94-73110
94 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 none
28-57787
28 days ago
28-57787
28 days ago
51-81907
51 days
22531 vasnesterov
author:vasnesterov
feat(Analysis): radius of convergence for `FormalMultilinearSeries.compContinuousLinearMap` - Add basic lemmas `compContinuousLinearMap_id` and `compContinuousLinearMap_comp`. - Prove lower and upper bounds for the convergence radius of `f.compContinuousLinearMap`. - Prove `radius_compNeg`: the convergence radii of `f(x)` and `f(-x)` are equal. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis 137/11 Mathlib/Analysis/Analytic/Basic.lean,Mathlib/Analysis/Analytic/CPolynomial.lean,Mathlib/Analysis/Analytic/Constructions.lean,Mathlib/Analysis/Calculus/FormalMultilinearSeries.lean,scripts/noshake.json 5 7 ['github-actions', 'j-loreaux', 'vasnesterov'] nobody none
28-7043
28 days ago
30-14317
30 days ago
95-9992
95 days
23497 chrisflav
author:chrisflav
chore(RingTheory/AdicCompletion/AsTensorProduct): golf using five lemma for modules --- - [x] depends on: #23496 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
30/81 Mathlib/RingTheory/AdicCompletion/AsTensorProduct.lean 1 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody none
27-75525
27 days ago
48-33482
1 month ago
48-34307
48 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 none
27-47902
27 days ago
27-56542
27 days ago
27-56596
27 days
24752 MichaelStollBayreuth
author:MichaelStollBayreuth
perf(Data.Real.Sqrt): make Real.sqrt irreducible We try to see what happens if we make `Real.sqrt` irreducible. There are cases where this makes unification *very* significantly faster, compare [#mathlib4 > Coercion triggers timeout @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Coercion.20triggers.20timeout/near/517177117). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data 1/0 Mathlib/Data/Real/Sqrt.lean 1 18 ['MichaelStollBayreuth', 'eric-wieser', 'github-actions', 'leanprover-bot'] nobody none
27-3829
27 days ago
29-17151
29 days ago
29-22628
29 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'] nobody none
26-49284
26 days ago
26-49291
26 days ago
26-49435
26 days
24872 smmercuri
author:smmercuri
feat: `apply` and `coe` results for `UniformSpace.Completion.mapRingHom` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology 9/0 Mathlib/Topology/Algebra/UniformRing.lean 1 1 ['github-actions'] nobody none
26-49063
26 days ago
26-49063
26 days ago
26-49111
26 days
24873 smmercuri
author:smmercuri
feat: `Subtype.map_ne` The restrictions to subtypes of two functions that never agree, also never agree. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data 7/0 Mathlib/Data/Subtype.lean 1 1 ['github-actions'] nobody none
26-48723
26 days ago
26-48725
26 days ago
26-48774
26 days
24883 madvorak
author:madvorak
chore(Data/Matrix): `Matrix.submatrix` naming convention I'm suggesting this change for the following reasons: (1) managing expectations — `r_reindex` looks more like a propositional argument at first glance (2) the original naming does not do justice to its motivation — there is nothing called `r` and `c` here — it would need to be `row_reindex` and `col_reindex` or something like that (if we wanted to use the convention for naming constants even tho we are naming a variable here) --- Old version: https://github.com/leanprover-community/mathlib4/pull/24135 t-data 11/11 Mathlib/Data/Matrix/ConjTranspose.lean,Mathlib/Data/Matrix/Defs.lean 2 1 ['github-actions'] nobody none
26-45358
26 days ago
26-45358
26 days ago
26-45348
26 days
24892 Ruben-VandeVelde
author:Ruben-VandeVelde
fix: add missing simps projections for ContinuousAddEquiv --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology 1/0 Mathlib/Topology/Algebra/ContinuousMonoidHom.lean 1 1 ['github-actions'] nobody none
26-36685
26 days ago
26-36687
26 days ago
26-36736
26 days
24889 Kha
author:Kha
chore: do not include cache requests in build benchmark 5/2 scripts/bench/temci-config.run.yml 1 4 ['Kha', 'github-actions', 'leanprover-bot'] nobody none
26-29277
26 days ago
26-39112
26 days ago
26-39095
26 days
22153 smmercuri
author:smmercuri
feat: weak approximation theorems for infinite places of a number field The number field $K$ is dense in $\prod_v (K, v)$ and in the infinite adele ring $\prod_v K_v$, where $v$ ranges over the infinite places, $(K, v)$ denotes $K$ equipped with the topology induced by $v$, and $K_v$ is the completion of $K$ at $v$. --- - [ ] depends on #22147 [![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$
543/2 Mathlib/Algebra/Order/AbsoluteValue/Basic.lean,Mathlib/Analysis/AbsoluteValue/Equivalence.lean,Mathlib/Analysis/Normed/Ring/WithAbs.lean,Mathlib/NumberTheory/NumberField/AdeleRing.lean,Mathlib/NumberTheory/NumberField/InfinitePlace/Basic.lean 5 1 ['github-actions'] nobody none
26-25905
26 days ago
26-43208
26 days ago
37-66790
37 days
24311 YaelDillies
author:YaelDillies
chore: replace `Monoid.IsTorsionFree` with `IsMulTorsionFree` From Toric --- - [x] depends on: #24312 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) toric t-algebra
label:t-algebra$
63/29 Mathlib/Algebra/Group/Torsion.lean,Mathlib/Combinatorics/Additive/CauchyDavenport.lean,Mathlib/GroupTheory/Order/Min.lean,Mathlib/GroupTheory/Torsion.lean,Mathlib/Topology/Instances/ZMultiples.lean 5 5 ['YaelDillies', 'b-mehta', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody none
26-24432
26 days ago
26-24432
26 days ago
26-37762
26 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 15 ['YaelDillies', 'eric-wieser', 'github-actions', 'j-loreaux', 'leanprover-community-bot-assistant', 'mathlib-bors'] nobody none
26-24175
26 days ago
26-24175
26 days ago
110-83611
110 days
24254 Louddy
author:Louddy
feat: valuation on RatFunc which is trivial on constants Given a valuation `v` on `RatFunc K` that is trivial on the constants `K`, the valuation on `RatFunc.X` determines to some degree the valuation on any `p : Polynomial K`. These are important in the context of Ostrowski's theorem for `RatFunc K`. Note that the condition that the valuation is trivial on constants is automatically fulfilled when `K` is finite. Co-authored-by: María Inés de Frutos Fernández <[mariaines.dff@gmail.com](mailto:mariaines.dff@gmail.com)> --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
66/0 Mathlib/FieldTheory/RatFunc/AsPolynomial.lean 1 29 ['Louddy', 'faenuccio', 'github-actions', 'mariainesdff'] nobody none
25-33991
25 days ago
25-34043
25 days ago
27-34964
27 days
18379 oeb25
author:oeb25
feat(Topology/ENNReal): Add `ENNReal.tsum_biUnion` This adds infinite versions of `Finset.sum_biUnion` to `ENNReal`s. --- One notable difference from the `Finset` version is that for `tsum` we have two ways for selecting the summands: `∑' x : ⋃ i ∈ S` or `∑' x : ⋃ i, t i`. This PR adds both. I tried to extend this beyond `ENNReal`, but didn't find a clean way to do it. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-topology 34/0 Mathlib/Data/Set/Lattice.lean,Mathlib/Data/Set/Pairwise/Lattice.lean,Mathlib/Topology/Instances/ENNReal/Lemmas.lean 3 12 ['github-actions', 'grunweg', 'j-loreaux', 'oeb25'] nobody none
25-33393
25 days ago
25-34406
25 days ago
127-82912
127 days
24730 YaelDillies
author:YaelDillies
feat(Bialgebra): group-like elements Define group-like elements in a bialgebra, ie units `a` such that `Δ a = a ⊗ₜ a`. We prove that group-like elements always form a group, and are linearly independent if the base ring is a domain. 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$
167/0 Mathlib.lean,Mathlib/RingTheory/Bialgebra/GroupLike.lean 2 18 ['YaelDillies', 'erdOne', 'eric-wieser', 'github-actions', 'leanprover-bot', 'mathlib4-dependent-issues-bot'] nobody none
25-15390
25 days ago
29-79464
29 days ago
29-81020
29 days
24891 YaelDillies
author:YaelDillies
feat: `M ≃ₗ[R] (Fin (Module.finrank R M) → R)` for `M` a finite `R`-module From Toric --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) toric t-algebra
label:t-algebra$
13/3 Mathlib/LinearAlgebra/Dimension/Free.lean,Mathlib/LinearAlgebra/FreeModule/Basic.lean,Mathlib/LinearAlgebra/FreeModule/Finite/Basic.lean 3 9 ['YaelDillies', 'erdOne', 'eric-wieser', 'github-actions'] nobody none
25-11279
25 days ago
26-21110
26 days ago
26-38032
26 days
22078 Louddy
author:Louddy
feat(SkewMonoidAlgebra): multiplication and algebraic instances # Multiplication and Algebraic Instances In this PR, we introduce the definition of the skewed convolution product on `SkewMonoidAlgebra k G`. Here, the product of two elements `f g : SkewMonoidAlgebra k G` is the finitely supported function whose value at `a` is the sum of `f x * (x • g y)` over all pairs `x, y` such that `x * y = a`. We also introduce the associated algebraic instances. ## Context This is the third part of a planned series of PRs aiming to formalise skew monoid algebras. The PRs are split to ease the review process. The moral sum of these planned PRs is #10541. The first and second part were #15878 and #19084. Co-authored-by: María Inés de Frutos Fernández <[mariaines.dff@gmail.com](mailto:mariaines.dff@gmail.com)> --- [![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$
453/45 Mathlib/Algebra/SkewMonoidAlgebra/Basic.lean 1 57 ['AntoineChambert-Loir', 'Louddy', 'github-actions', 'kbuzzard'] nobody none
24-42459
24 days ago
26-39366
26 days ago
98-59896
98 days
24948 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/) t-combinatorics 91/0 Mathlib/Combinatorics/SimpleGraph/Bipartite.lean 1 1 ['github-actions'] nobody none
24-40626
24 days ago
24-40631
24 days ago
24-40679
24 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 65/48 Mathlib/Analysis/Analytic/OfScalars.lean,Mathlib/Analysis/Oscillation.lean,Mathlib/Data/Finset/Lattice/Fold.lean,Mathlib/Data/Finset/Max.lean,Mathlib/LinearAlgebra/Eigenspace/Triangularizable.lean,Mathlib/MeasureTheory/Integral/Lebesgue/Countable.lean,Mathlib/MeasureTheory/Measure/LevyProkhorovMetric.lean,Mathlib/Order/Interval/Basic.lean,Mathlib/Order/Interval/Set/WithBotTop.lean,Mathlib/Order/WithBot.lean,Mathlib/Probability/Moments/Variance.lean,Mathlib/RingTheory/PowerBasis.lean,Mathlib/Topology/MetricSpace/Holder.lean,Mathlib/Topology/MetricSpace/HolderNorm.lean 14 20 ['YaelDillies', 'b-mehta', 'eric-wieser', 'github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'urkud'] nobody none
23-44302
23 days ago
23-44323
23 days ago
73-36877
73 days
24967 vasnesterov
author:vasnesterov
perf(Topology/Metrizable): lower `IsCompletelyMetrizableSpace.MetrizableSpace` priority The priority of `IsCompletelyMetrizableSpace.MetrizableSpace` was set to 100, causing it to be applied before `EMetricSpace.metrizableSpace` and leading to wasted time trying to infer completeness. This PR sets it to 90. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology easy 1/1 Mathlib/Topology/Metrizable/CompletelyMetrizable.lean 1 4 ['github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot'] nobody none
23-30787
23 days ago
23-69878
23 days ago
23-71889
23 days
22739 joelriou
author:joelriou
feat(CategoryTheory/Abelian): isomorphisms modulo a Serre class --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory 192/0 Mathlib.lean,Mathlib/CategoryTheory/Abelian/SerreClass/MorphismProperty.lean,Mathlib/CategoryTheory/Limits/Shapes/Equalizers.lean,Mathlib/CategoryTheory/Limits/Shapes/Kernels.lean,Mathlib/CategoryTheory/Preadditive/Basic.lean 5 7 ['TwoFX', 'erdOne', 'github-actions', 'joelriou'] nobody none
23-22640
23 days ago
23-22640
23 days ago
81-8568
81 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 none
22-38855
22 days ago
38-38495
1 month ago
38-46410
38 days
24191 joelriou
author:joelriou
refactor(CategoryTheory): redefine triangulated subcategories using ObjectProperty --- - [x] depends on: #22574 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory 279/191 Mathlib/Algebra/Homology/DerivedCategory/Basic.lean,Mathlib/CategoryTheory/ObjectProperty/ContainsZero.lean,Mathlib/CategoryTheory/ObjectProperty/Shift.lean,Mathlib/CategoryTheory/Triangulated/HomologicalFunctor.lean,Mathlib/CategoryTheory/Triangulated/Subcategory.lean 5 5 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody none
22-30674
22 days ago
28-3496
28 days ago
46-67686
46 days
24960 linesthatinterlace
author:linesthatinterlace
feat(Data/Finite/PermOf): Add an array-based implementation of finite permutations, `PermOf`. Implements `PermOf`, an array-based implementation of finite permutations/ --- As part of my PhD, I created this implementation. I have more to add to it, but I'm making this relatively small initial commit to exhibit the core definitions before I start building anything elaborate. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data 378/0 Mathlib.lean,Mathlib/Data/Finite/PermLT/Defs.lean,Mathlib/Data/Finite/PermLT/Group.lean,Mathlib/Data/Finite/PermLT/MulAction.lean 4 35 ['eric-wieser', 'github-actions', 'linesthatinterlace'] nobody none
22-7695
22 days ago
24-19913
24 days ago
24-19968
24 days
24966 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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-differential-geometry 154/13 Mathlib/Geometry/Manifold/PartitionOfUnity.lean 1 3 ['github-actions', 'grunweg', 'michaellee94'] nobody none
21-79963
21 days ago
23-17943
23 days ago
23-45496
23 days
21522 riccardobrasca
author:riccardobrasca
feat: add Mathlib.RingTheory.DedekindDomain.Instances We add a new file `Mathlib.RingTheory.DedekindDomain.Instances` containing various instances that are useful to work with the localization a prime of an extension of Dedekind domains. As a practical example we golf a tedious proof in `Mathlib.RingTheory.Ideal/Norm.RelNorm` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-algebra
label:t-algebra$
253/71 Mathlib.lean,Mathlib/RingTheory/DedekindDomain/Different.lean,Mathlib/RingTheory/DedekindDomain/Instances.lean,Mathlib/RingTheory/DedekindDomain/IntegralClosure.lean,Mathlib/RingTheory/Ideal/Norm/RelNorm.lean,Mathlib/RingTheory/IntegralClosure/IntegralRestrict.lean,Mathlib/RingTheory/Localization/AtPrime.lean,Mathlib/RingTheory/Localization/Basic.lean,Mathlib/RingTheory/Localization/LocalizationLocalization.lean,Mathlib/RingTheory/RingHom/Finite.lean,Mathlib/RingTheory/Trace/Quotient.lean 11 34 ['YaelDillies', 'erdOne', 'fpvandoorn', 'github-actions', 'riccardobrasca'] nobody none
21-26828
21 days ago
26-26297
26 days ago
92-58869
92 days
24719 madvorak
author:madvorak
feat(LinearAlgebra/Matrix/NonsingularInverse): inverting `Matrix` inverts its `LinearEquiv` --- Discussion: https://leanprover.zulipchat.com/#narrow/channel/144837-PR-reviews/topic/.2324719.20cannot.20find.20home/with/517142655 t-algebra
label:t-algebra$
10/0 Mathlib/LinearAlgebra/Matrix/NonsingularInverse.lean 1 11 ['eric-wieser', 'github-actions', 'madvorak'] nobody none
21-20152
21 days ago
29-24997
29 days ago
30-61226
30 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 none
21-9651
21 days ago
21-9775
21 days ago
21-13240
21 days
25036 Parcly-Taxel
author:Parcly-Taxel
feat: IMO 2001 Q4 IMO 131/4 Archive.lean,Archive/Imo/Imo2001Q4.lean,Mathlib/Logic/Equiv/Fin/Rotate.lean 3 1 ['github-actions'] nobody none
20-51766
20 days ago
20-52508
20 days ago
20-52492
20 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$
215/155 Mathlib/Algebra/Algebra/Operations.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Affine/Point.lean,Mathlib/RingTheory/Extension/Basic.lean,Mathlib/RingTheory/Finiteness/Basic.lean,Mathlib/RingTheory/Finiteness/Ideal.lean,Mathlib/RingTheory/HopkinsLevitzki.lean,Mathlib/RingTheory/Ideal/Maps.lean,Mathlib/RingTheory/Ideal/Operations.lean 8 7 ['alreadydone', 'github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody none
20-38962
20 days ago
20-39117
20 days ago
97-8246
97 days
20160 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/) t-data 69/0 Mathlib/Data/Seq/Seq.lean 1 3 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody none
20-37866
20 days ago
27-81161
27 days ago
27-81310
27 days
22631 Thmoas-Guan
author:Thmoas-Guan
feat(Algebra): define associated graded structure for abelian group In this PR we define the associated graded structure for abelian group when given a filtration and only give some basic lemmas about it. Further results would be given in #20913 --- - [x] depends on: #24071 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
155/0 Mathlib.lean,Mathlib/RingTheory/FilteredAlgebra/AssociatedGraded.lean 2 17 ['AntoineChambert-Loir', 'Thmoas-Guan', 'eric-wieser', 'github-actions', 'kbuzzard', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody none
20-35308
20 days ago
20-35328
20 days ago
94-79909
94 days
25044 alreadydone
author:alreadydone
feat(Topology/Algebra): `Homeomorph` version of `unitsEquivNeZero` also add `Topology.IsEmbedding.homeomorphImage`: a set is homeomorphic to its image under any embedding. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-topology
label:t-algebra$
51/28 Mathlib/Topology/Algebra/GroupWithZero.lean,Mathlib/Topology/Homeomorph/Lemmas.lean 2 1 ['github-actions'] nobody none
20-28054
20 days ago
20-32309
20 days ago
20-32293
20 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 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody none
20-10483
20 days ago
20-18238
20 days ago
20-19618
20 days
24928 kim-em
author:kim-em
chore: remove some `Nat` shortcut instances t-data 0/9 Mathlib/Algebra/Ring/Divisibility/Basic.lean,Mathlib/Data/List/TakeDrop.lean,Mathlib/Data/Nat/Basic.lean 3 10 ['Ruben-VandeVelde', 'github-actions', 'kim-em', 'leanprover-bot', 'leanprover-community-mathlib4-bot'] nobody none
19-67618
19 days ago
19-67618
19 days ago
25-43867
25 days
25068 Parcly-Taxel
author:Parcly-Taxel
feat: IMO 2001 Q3 IMO 111/0 Archive.lean,Archive/Imo/Imo2001Q3.lean 2 1 ['github-actions'] nobody none
19-64371
19 days ago
19-67128
19 days ago
19-67112
19 days
24931 qawbecrdtey
author:qawbecrdtey
feat(Data/Nat/Sqrt): Added lemma `Nat.add_one_sqrt_le_of_pos` --- This commit proves a single lemma `Nat.add_one_sqrt_le_of_pos`. ```lean lemma add_one_sqrt_le_of_pos {n : ℕ} (hn : 1 ≤ n) : (n + 1).sqrt ≤ n ``` [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data easy 7/0 Mathlib/Data/Nat/Sqrt.lean 1 4 ['Ruben-VandeVelde', 'eric-wieser', 'github-actions', 'qawbecrdtey'] nobody none
19-23003
19 days ago
25-37853
25 days ago
25-37911
25 days
24703 robin-carlier
author:robin-carlier
feat(CategoryTheory/Monoidal): external product of diagrams in monoidal categories Given functors `K₁ : J₁ ⥤ C` and `K₂ : J₂ ⥤ C` with values in a monoidal category, define a construction `externalProduct K₁ K₂` (denoted `K₁ ⊠ K₂`) as the bifunctor `(j₁, j₂) ↦ K₁ j₁ ⊗ K₂ j₂`. We show that composition of this construction with the diagonal functor to the product recovers the pointwise tensor product of functors, and we show that this construction satisfies a symmetry whenever `C` is braided. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory 99/0 Mathlib.lean,Mathlib/CategoryTheory/Monoidal/ExternalProduct.lean 2 5 ['github-actions', 'joelriou'] nobody none
18-47098
18 days ago
18-47161
18 days ago
31-2826
31 days
25101 erdOne
author:erdOne
feat(AlgebraicGeometry): building morphisms into Proj --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebraic-geometry 231/3 Mathlib/AlgebraicGeometry/ProjectiveSpectrum/Basic.lean,Mathlib/AlgebraicGeometry/Restrict.lean,Mathlib/AlgebraicGeometry/Scheme.lean,Mathlib/RingTheory/GradedAlgebra/HomogeneousLocalization.lean 4 6 ['erdOne', 'github-actions', 'joelriou'] nobody none
17-78571
17 days ago
17-78571
17 days ago
18-58260
18 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'] nobody none
17-68079
17 days ago
17-68079
17 days ago
17-68132
17 days
25124 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 1 ['github-actions'] nobody none
17-63123
17 days ago
17-65948
17 days ago
17-65991
17 days
24485 dagurtomas
author:dagurtomas
feat(CategoryTheory): localization preserves braided structure --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory 733/427 Mathlib.lean,Mathlib/CategoryTheory/Localization/Monoidal.lean,Mathlib/CategoryTheory/Localization/Monoidal/Basic.lean,Mathlib/CategoryTheory/Localization/Monoidal/Braided.lean,Mathlib/CategoryTheory/Monoidal/Braided/Basic.lean,Mathlib/CategoryTheory/Sites/Monoidal.lean 6 7 ['dagurtomas', 'github-actions', 'joelriou', 'leanprover-community-bot-assistant'] nobody none
17-41565
17 days ago
17-41565
17 days ago
27-82564
27 days
24651 Hagb
author:Hagb
feat(RingTheory/Finiteness/Defs): span of a set is finitely generated iff generated by a finite subset --- - [ ] depends on: #24648 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra
label:t-algebra$
14/0 Mathlib/RingTheory/Finiteness/Defs.lean 1 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody none
17-38635
17 days ago
17-38654
17 days ago
17-43206
17 days
23365 vasnesterov
author:vasnesterov
feat(Tactic/Simproc): nested quantifiers in `existsAndEq` Generalize the `existsAndEq` simproc to nested existential quantifiers. For example `∃ a, p a ∧ ∃ b, a = f b ∧ q b` now simplifies to `∃ b, p (f b) ∧ q b`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-meta 440/73 Mathlib/Tactic/Simproc/ExistsAndEq.lean,MathlibTest/Simproc/ExistsAndEq.lean 2 41 ['JovanGerb', 'b-mehta', 'eric-wieser', 'github-actions', 'grunweg', 'kim-em', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'vasnesterov'] nobody none
17-36555
17 days ago
67-74040
2 months ago
73-14281
73 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'] nobody none
17-25545
17 days ago
17-25612
17 days ago
34-10636
34 days
22931 chrisflav
author:chrisflav
refactor(RingTheory/RingHom): factor out proofs for `Algebra.FiniteType` 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.FiniteType` 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: #22933 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
126/119 Mathlib/RingTheory/FiniteType.lean,Mathlib/RingTheory/RingHom/Finite.lean,Mathlib/RingTheory/RingHom/FiniteType.lean 3 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody none
17-23901
17 days ago
17-25275
17 days ago
17-26487
17 days
25112 linesthatinterlace
author:linesthatinterlace
feat(`Algebra/Group/Prod`): Add API for inclusion and projection maps from and to the product of units. Adds API for inclusion and projection maps from and to the product of units. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
99/30 Mathlib/Algebra/BigOperators/Associated.lean,Mathlib/Algebra/Group/Prod.lean,Mathlib/Data/Nat/Totient.lean,Mathlib/Topology/Algebra/Group/Basic.lean 4 9 ['eric-wieser', 'github-actions', 'linesthatinterlace', 'pechersky'] nobody none
17-23021
17 days ago
18-25288
18 days ago
18-25451
18 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'] nobody none
17-16885
17 days ago
19-63787
19 days ago
19-63844
19 days
25071 erdOne
author:erdOne
feat(EllipticCurve): basic API for singular cubics --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebraic-geometry 320/0 Mathlib.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Singular/Basic.lean,Mathlib/AlgebraicGeometry/EllipticCurve/VariableChange.lean 3 34 ['Multramate', 'acmepjz', 'erdOne', 'github-actions'] nobody none
16-60121
16 days ago
19-61944
19 days ago
19-62000
19 days
23312 xroblot
author:xroblot
feat(NumberField/Units): prove that a family of units is of max rank iff its closure has finite index Let `u : Fin (rank K) → (𝓞 K)ˣ` be a family of units of a number field `K`. We prove that `isMaxRank u`, that is its regulator is nonzero, iff `closure (Set.range u))` has finite index. --- - [x] depends on: #22882 - [x] depends on: #23063 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-number-theory 70/3 Mathlib/GroupTheory/Index.lean,Mathlib/LinearAlgebra/FreeModule/Finite/Quotient.lean,Mathlib/NumberTheory/NumberField/Units/Regulator.lean 3 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody none
16-25473
16 days ago
16-25491
16 days ago
16-26436
16 days
25150 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/) t-category-theory 191/0 Mathlib.lean,Mathlib/CategoryTheory/Bicategory/LocallyGroupoid.lean 2 1 ['github-actions'] nobody none
16-15580
16 days ago
16-19133
16 days ago
16-19188
16 days
21103 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`. --- - [x] depends on: #21098 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory 118/5 Mathlib/AlgebraicTopology/SimplexCategory/Basic.lean,Mathlib/AlgebraicTopology/SimplicialSet/Degenerate.lean 2 5 ['dagurtomas', 'gio256', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody none
15-86359
15 days ago
51-83505
1 month ago
90-28708
90 days
25157 wwylele
author:wwylele
feat(Data/Real): add embedding of archimedean groups into Real This is part of #25140, and is the special case of Hahn embedding theorem applied to archimedean group. The construction is rather unpleasant as it uses explicit Cauchy sequence with essentially the binary representation of numbers, but I haven't found a better way to do this. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data 288/0 Mathlib.lean,Mathlib/Data/Real/Embedding.lean 2 3 ['eric-wieser', 'github-actions', 'wwylele'] nobody none
15-74090
15 days ago
16-11777
16 days ago
16-11830
16 days
25105 erdOne
author:erdOne
feat(AlgebraicGeometry): inverse limit of nonempty quasicompact closeds is nonempty --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-algebraic-geometry 92/2 Mathlib/AlgebraicGeometry/AffineTransitionLimit.lean,Mathlib/AlgebraicGeometry/Morphisms/Separated.lean,Mathlib/CategoryTheory/Comma/Over/Basic.lean 3 1 ['github-actions'] nobody none
15-64061
15 days ago
18-42130
18 days ago
18-42182
18 days
24819 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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
27/3 Mathlib/RingTheory/MvPolynomial/Groebner.lean 1 4 ['Hagb', 'github-actions'] nobody none
15-12814
15 days ago
28-6092
28 days ago
28-6144
28 days
21283 erdOne
author:erdOne
feat: topology on Hom(R, S) in `CommRingCat` Co-authored-by: Christian Merten --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-topology
label:t-algebra$
239/0 Mathlib.lean,Mathlib/Algebra/Category/Ring/Constructions.lean,Mathlib/Algebra/Category/Ring/Topology.lean,Mathlib/RingTheory/TensorProduct/Basic.lean,Mathlib/Topology/Constructions.lean,Mathlib/Topology/Homeomorph/Lemmas.lean,scripts/noshake.json 7 21 ['dagurtomas', 'erdOne', 'github-actions', 'kbuzzard'] nobody none
15-7653
15 days ago
27-12564
27 days ago
109-40479
109 days
24103 plp127
author:plp127
feat(Topology/UniformSpace/OfCompactT2): generalize theorem Generalize `uniformSpaceOfCompactT2` to `uniformSpaceOfCompactR1`. --- - [ ] depends on: #24098 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology 48/24 Mathlib/Topology/Separation/Regular.lean,Mathlib/Topology/UniformSpace/OfCompactT2.lean 2 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody none
15-3140
15 days ago
15-3162
15 days ago
46-79521
46 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 14 ['YaelDillies', 'erdOne', 'eric-wieser', 'github-actions'] nobody none
15-2432
15 days ago
15-2493
15 days ago
15-6417
15 days
23368 b-reinke
author:b-reinke
feat(GroupTheory/FreeGroup/ReducedWords): add theory of reduced words Upstreamed from the [EquationalTheories](https://github.com/teorth/equational_theories) project. This PR adds the file `GroupTheory/FreeGroup/ReducedWords.lean`, where the predicate of reduced words is defined. It is shown that `reduce` and `toWord` produce reduced words. This is done in preparation for the theory of cyclically reduced words. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-geometric-group-theory t-algebra
label:t-algebra$
104/0 Mathlib.lean,Mathlib/GroupTheory/FreeGroup/ReducedWords.lean 2 37 ['b-reinke', 'github-actions', 'tb65536', 'vlad902'] nobody 2
14-59970
14 days ago
74-25781
2 months ago
74-33611
74 days
25188 vlad902
author:vlad902
feat: add lemmas about `List.scanr` I add basic lemmas to reason about `List.scanr`, and slightly clean-up the file and add some basic lemmas to keep the API unified with the one for `List.scanl`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data 84/18 Mathlib/Data/List/Scan.lean 1 5 ['b-mehta', 'github-actions', 'vlad902'] nobody 1
14-48841
14 days ago
14-49069
14 days ago
14-72569
14 days
25204 YaelDillies
author:YaelDillies
refactor: redefine `ProperCone` as an `abbrev` for `ClosedSubmodule` ... and derive the `ProperCone` operations from `ClosedSubmodule` too. Also rename the scalar ring from `𝕜` to `R`. From Toric --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) toric t-analysis 79/90 Mathlib/Analysis/Convex/Cone/Proper.lean 1 1 ['github-actions'] nobody none
14-37093
14 days ago
14-37135
14 days ago
14-37146
14 days
25209 upobir
author:upobir
feat(NumberTheory/Divisors): add int divisors --- this PR adds `Int.divisors` analogous to `Nat.divisors`. Some preliminary results are proven for the new definition. Imports have also been modified by using `#min_imports` [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-number-theory 125/4 Mathlib/NumberTheory/Divisors.lean 1 8 ['Paul-Lez', 'eric-wieser', 'github-actions', 'upobir'] nobody none
14-18151
14 days ago
14-24775
14 days ago
14-24832
14 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 none
14-10564
14 days ago
55-85262
1 month ago
55-85314
55 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 none
14-1019
14 days ago
19-63820
19 days ago
19-63817
19 days
23848 emilyriehl
author:emilyriehl
feat(AlgebraicTopology/SimplicialSet/NerveAdjunction): to Strict Segal 2 Under a suitable hypothesis, a map of 2-truncated simplicial sets can be generated from a refl prefunctor between the underlying reflexive quivers --- provided the codomain is `StrictSegal`. This abstracts a previously formalized result that requires the codomain to be the 2-truncated nerve of a category. Co-authored-by: Aaron Liu --- The current draft displays the old code for comparison with new versions labeled ALT. After initial review this will be cut. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) infinity-cosmos t-topology t-category-theory 490/202 Mathlib/AlgebraicTopology/SimplexCategory/Basic.lean,Mathlib/AlgebraicTopology/SimplicialSet/HomotopyCat.lean,Mathlib/AlgebraicTopology/SimplicialSet/NerveAdjunction.lean,Mathlib/AlgebraicTopology/SimplicialSet/StrictSegal.lean,Mathlib/CategoryTheory/ComposableArrows.lean,Mathlib/CategoryTheory/EqToHom.lean 6 17 ['emilyriehl', 'github-actions', 'joelriou'] nobody none
13-65658
13 days ago
20-7827
20 days ago
26-75823
26 days
25182 YaelDillies
author:YaelDillies
feat: `(M →* N₁) ≃* (M →* N₂)` if `N₁ ≃* N₂` From Toric --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) toric t-algebra
label:t-algebra$
63/12 Mathlib/Algebra/Category/Grp/ForgetCorepresentable.lean,Mathlib/Algebra/Category/Grp/LargeColimits.lean,Mathlib/Algebra/Category/MonCat/ForgetCorepresentable.lean,Mathlib/Algebra/Group/Equiv/Basic.lean,Mathlib/GroupTheory/FiniteAbelian/Duality.lean 5 10 ['YaelDillies', 'eric-wieser', 'github-actions'] nobody none
13-48712
13 days ago
14-41952
14 days ago
15-32593
15 days
21745 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/) large-import t-topology t-category-theory 253/7 Mathlib/AlgebraicTopology/SimplexCategory/GeneratorsRelations/NormalForms.lean 1 21 ['dagurtomas', 'github-actions', 'joelriou', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'robin-carlier'] nobody none
13-47257
13 days ago
25-41685
25 days ago
48-49632
48 days
25240 IvanRenison
author:IvanRenison
feat(Analysis/InnerProductSpace/Projection): add lemma `Submodule.le_iff_orthogonal_le_orthogonal` and similars --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis 25/0 Mathlib/Analysis/InnerProductSpace/Projection.lean 1 1 ['github-actions'] nobody none
13-15930
13 days ago
13-15933
13 days ago
13-15986
13 days
23684 alreadydone
author:alreadydone
feat(RingTheory): integral extensions of comm. rings are local homs --- The import increase only affects one file so I hope it's okay. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-algebra
label:t-algebra$
57/65 Mathlib/Algebra/Field/Equiv.lean,Mathlib/Algebra/Group/Invertible/Basic.lean,Mathlib/Algebra/GroupWithZero/Units/Basic.lean,Mathlib/AlgebraicGeometry/Morphisms/Proper.lean,Mathlib/FieldTheory/LinearDisjoint.lean,Mathlib/LinearAlgebra/Dimension/Localization.lean,Mathlib/RingTheory/Artinian/Ring.lean,Mathlib/RingTheory/IntegralClosure/Algebra/Defs.lean,Mathlib/RingTheory/IntegralClosure/IsIntegralClosure/Basic.lean,Mathlib/RingTheory/LinearDisjoint.lean,Mathlib/RingTheory/Localization/FractionRing.lean,Mathlib/RingTheory/Localization/Integral.lean,Mathlib/RingTheory/SimpleRing/Field.lean 13 4 ['alreadydone', 'github-actions', 'xroblot'] nobody 1
13-6805
13 days ago
65-72197
2 months ago
65-72217
65 days
25224 xcloudyunx
author:xcloudyunx
feat(Combinatorics/SimpleGraph): edgeSet of Eulerian walk equal to edgeSet of graph --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-combinatorics easy 6/0 Mathlib/Combinatorics/SimpleGraph/Trails.lean 1 2 ['IvanRenison', 'github-actions'] nobody none
12-83709
12 days ago
13-74712
13 days ago
13-75614
13 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'] nobody none
12-83102
12 days ago
13-74514
13 days ago
13-74571
13 days
25248 xcloudyunx
author:xcloudyunx
feat(Combinatorics/SimpleGraph): Add Subgraph.inclusion_edge_apply_coe and inclusion_edgeSet_apply_coe --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-combinatorics 12/0 Mathlib/Combinatorics/SimpleGraph/Subgraph.lean 1 1 ['github-actions'] nobody none
12-76744
12 days ago
12-76745
12 days ago
12-76800
12 days
25238 Hagb
author:Hagb
feat(Tactic/ComputeDegree): add support for scalar multiplication with different types It would be able to deal with `a • (X : R[X])` where `a : S` is in a different type `S` with `[SMulZeroClass S R]`. --- - [x] depends on: #25237 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor 17/5 Mathlib/Tactic/ComputeDegree.lean,MathlibTest/ComputeDegree.lean 2 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody none
12-56734
12 days ago
12-81177
12 days ago
12-83080
12 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 none
12-48292
12 days ago
16-14031
16 days ago
16-14015
16 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 7 ['Parcly-Taxel', 'YaelDillies', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant'] nobody 1
12-45087
12 days ago
12-45105
12 days ago
59-44919
59 days
25253 Ruben-VandeVelde
author:Ruben-VandeVelde
feat: add AlgHom.natCard_of_splits --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 21/7 Mathlib/FieldTheory/PrimitiveElement.lean,Mathlib/FieldTheory/Separable.lean,Mathlib/SetTheory/Cardinal/Finite.lean 3 1 ['github-actions'] nobody none
12-43025
12 days ago
12-43107
12 days ago
12-43091
12 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 none
12-42970
12 days ago
13-18912
13 days ago
19-23308
19 days
25179 YaelDillies
author:YaelDillies
feat: `#track_sorry`, a command to find usage of `sorry` `#track_sorry foo` returns a non-sorry-free declaration `bar` which `foo` depends on, if such `bar` exists. Such a command is a recurrent need of the community, see eg [here](https://leanprover.zulipchat.com/#narrow/channel/217875-Is-there-code-for-X.3F/topic/Hunting.20down.20axioms/with/495448595) most recently. From Toric Co-authored-by: Henrik Böving --- An alternative implementation was provided in [#Is there code for X? > ✔ Finding usages of `sorry` in external code @ 💬](https://leanprover.zulipchat.com/#narrow/channel/217875-Is-there-code-for-X.3F/topic/.E2.9C.94.20Finding.20usages.20of.20.60sorry.60.20in.20external.20code/near/430509619) by @kmill. I prefer the current one because it only prints something for uses of `sorry` and not the other three standard axioms. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) toric t-meta 71/0 Mathlib.lean,Mathlib/Util/TrackSorry.lean 2 11 ['YaelDillies', 'eric-wieser', 'github-actions', 'kmill'] nobody none
12-33079
12 days ago
15-41894
15 days ago
15-41948
15 days
25257 Hagb
author:Hagb
feat(Mathlib/Algebra/Polynomial/Degree/Domain.lean): generalize `natDegree_smul` from `SMulWithZero` to `SMulZeroClass` as suggested by @eric-wieser in https://github.com/leanprover-community/mathlib4/pull/25237#discussion_r2111599865 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra
label:t-algebra$
4/3 Mathlib/Algebra/Polynomial/Degree/Domain.lean 1 1 ['github-actions'] nobody none
12-26109
12 days ago
12-26109
12 days ago
12-26171
12 days
25262 Ruben-VandeVelde
author:Ruben-VandeVelde
chore: add missing deprecations From #23643, #23804, #24762, #24827, #24833, and #25016. --- Maybe for some of those there could be reasons to argue that a deprecation is not terribly useful, but adding them is so cheap that I don't think it's worth spending much time arguing about it. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 36/0 Mathlib/AlgebraicGeometry/IdealSheaf/Basic.lean,Mathlib/Analysis/SpecialFunctions/Complex/LogBounds.lean,Mathlib/Analysis/SpecialFunctions/MulExpNegMulSqIntegral.lean,Mathlib/GroupTheory/Perm/Finite.lean,Mathlib/GroupTheory/Perm/Support.lean,Mathlib/NumberTheory/NumberField/InfinitePlace/TotallyRealComplex.lean,Mathlib/RingTheory/Ideal/Operations.lean,Mathlib/RingTheory/MvPowerSeries/PiTopology.lean 8 1 ['github-actions'] nobody none
12-15004
12 days ago
12-17260
12 days ago
12-17244
12 days
25251 YaelDillies
author:YaelDillies
chore: move pointed cones, proper cones Pointed cones too are a kind of algebraic cone. They therefore move to the new `Geometry.Convex.Cone` folder. In turn, this makes proper cones the primitive kind of topological/analytic cones, and therefore `Analysis.Convex.Cone.Proper` gets renamed to `Analysis.Convex.Cone.Basic`. The two sections about dual pointed cones and dual proper cones move to the existing `Analysis.Convex.Cone.InnerDual`. The READMEs about `Geometry.Convex.Cone` and `Analysis.Convex.Cone` get updated to reflect that the separation is non-topology vs topology, rather topology vs analysis. From Toric --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) file-removed toric large-import t-analysis 112/115 Mathlib.lean,Mathlib/Analysis/Convex/Cone/Basic.lean,Mathlib/Analysis/Convex/Cone/Closure.lean,Mathlib/Analysis/Convex/Cone/InnerDual.lean,Mathlib/Analysis/Convex/Cone/README.md,Mathlib/Geometry/Convex/Cone/Basic.lean,Mathlib/Geometry/Convex/Cone/Pointed.lean,Mathlib/Geometry/Convex/Cone/README.md 8 2 ['github-actions', 'leanprover-community-bot-assistant'] nobody none
12-12573
12 days ago
12-20075
12 days ago
12-36173
12 days
25266 j-loreaux
author:j-loreaux
feat: add path component of the identity in a locally path connected topological group, as an open normal subgroup --- From [LeanOA](https://github.com/j-loreaux/LeanOA) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology 101/8 Mathlib.lean,Mathlib/Topology/Connected/PathComponentOne.lean,Mathlib/Topology/Connected/PathConnected.lean,Mathlib/Topology/Path.lean 4 1 ['github-actions'] nobody none
12-7869
12 days ago
12-10701
12 days ago
12-11347
12 days
25271 YaelDillies
author:YaelDillies
feat: promote an `AlgEquiv` preserving `counit` and `comul` to a `BialgEquiv` From Toric --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) toric t-algebra
label:t-algebra$
38/24 Mathlib/Algebra/Algebra/Equiv.lean,Mathlib/Algebra/Algebra/Hom.lean,Mathlib/RingTheory/Bialgebra/Equiv.lean 3 1 ['github-actions'] nobody none
12-6409
12 days ago
12-10058
12 days ago
12-10053
12 days
25173 Timeroot
author:Timeroot
"Junk value" test file Add to MathlibTest a file that documents junk values of many functions, and explains some of their motivations and gotchas. --- Based on the conversation [on Zulip](https://leanprover.zulipchat.com/#narrow/channel/113488-general/topic/Documenting.20lean.20pitfalls.3A.20feedback.20requested/near/520155520). [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 362/2 Mathlib/Data/Nat/Find.lean,MathlibTest/Junk.lean 2 15 ['Timeroot', 'github-actions', 'plp127'] nobody none
11-84537
11 days ago
15-59398
15 days ago
15-59382
15 days
24582 pechersky
author:pechersky
feat(GroupTheory/ArchimedeanDensely): Unique (ℤ ≃+o ℤ) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) - [x] depends on: #24580 t-order t-algebra
label:t-algebra$
44/0 Mathlib/Data/Int/Cast/Lemmas.lean,Mathlib/GroupTheory/ArchimedeanDensely.lean 2 5 ['eric-wieser', 'github-actions', 'mathlib4-dependent-issues-bot', 'pechersky'] nobody none
11-65302
11 days ago
11-65375
11 days ago
15-28500
15 days
25273 YaelDillies
author:YaelDillies
feat: `Finsupp.linearCombination MonoidAlgebra.of = id` From Toric --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-algebra
label:t-algebra$
8/1 Mathlib/Algebra/MonoidAlgebra/Defs.lean 1 4 ['YaelDillies', 'eric-wieser', 'github-actions'] nobody none
11-40091
11 days ago
12-8231
12 days ago
12-8280
12 days
25291 YaelDillies
author:YaelDillies
chore(Geometry/Convex/Cone/Basic): clean up Rename all the `ConvexCone`s in the file to `C`, `C₁`, `C₂`. Previously they were `S`, `T`, `K₁`, `K₂`. Make sure to tag all the relevant lemmas with `norm_cast`. Fix lemma names. Golf proofs. From Toric --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-convex-geometry toric 145/186 Mathlib/Analysis/Convex/Cone/Pointed.lean,Mathlib/Geometry/Convex/Cone/Basic.lean 2 1 ['github-actions'] nobody none
11-36836
11 days ago
11-41271
11 days ago
11-41327
11 days
22490 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. --- - [x] depends on: #22474 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory 160/0 Mathlib.lean,Mathlib/CategoryTheory/Functor/Derived/PointwiseRightDerived.lean 2 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody none
11-8730
11 days ago
11-8995
11 days ago
11-11016
11 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 none
11-7081
11 days ago
11-7081
11 days ago
11-25466
11 days
25062 erdOne
author:erdOne
feat(Algebra/MvPolynomial): nilpotents and units --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
113/0 Mathlib.lean,Mathlib/Algebra/MvPolynomial/Nilpotent.lean,Mathlib/Data/Finsupp/Basic.lean 3 8 ['alreadydone', 'erdOne', 'eric-wieser', 'github-actions'] nobody none
10-22453
10 days ago
19-70059
19 days ago
19-70108
19 days
24689 chrisflav
author:chrisflav
feat(Topology): compact open covered sets This is used to define the fpqc topology for schemes. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) maintainer-merge t-algebraic-geometry t-topology 219/0 Mathlib.lean,Mathlib/Data/Set/Sigma.lean,Mathlib/Topology/Compactness/Compact.lean,Mathlib/Topology/Sets/CompactOpenCovered.lean,Mathlib/Topology/Sets/Opens.lean,Mathlib/Topology/Spectral/Prespectral.lean 6 5 ['chrisflav', 'erdOne', 'github-actions', 'leanprover-community-bot-assistant'] nobody none
10-5014
10 days ago
10-5399
10 days ago
31-65140
31 days
25313 jt496
author:jt496
feat(SimpleGraph/FiveWheelLike): add the Andrásfai-Erdős-Sós theorem Add the Andrásfai-Erdős-Sós theorem `colorable_of_cliqueFree_lt_minDegree` which says that an `r + 1`-cliquefree graph `G` with sufficiently large minimum degree is `r`-colorable. Co-authored-by: Lian Bremner Tattersall --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-combinatorics 307/4 Mathlib/Combinatorics/SimpleGraph/FiveWheelLike.lean 1 1 ['github-actions'] nobody none
9-73651
9 days ago
10-35687
10 days ago
10-35738
10 days
21950 erdOne
author:erdOne
feat(NumberTheory/Padics): the completion of `ℚ` at a finite place is `ℚ_[p]` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-number-theory 253/1 Mathlib.lean,Mathlib/Algebra/GroupWithZero/WithZero.lean,Mathlib/NumberTheory/Padics/HeightOneSpectrum.lean,Mathlib/NumberTheory/Padics/PadicNumbers.lean,Mathlib/Topology/Algebra/Valued/WithVal.lean,Mathlib/Topology/Algebra/WithZeroMulInt.lean,Mathlib/Topology/Algebra/WithZeroTopology.lean 7 22 ['Ruben-VandeVelde', 'erdOne', 'github-actions', 'leanprover-community-bot-assistant', 'pechersky', 'smmercuri', 'xroblot'] nobody 1
9-68894
9 days ago
9-68894
9 days ago
51-21490
51 days
25322 thorimur
author:thorimur
style: use simplex notation (`⦋n⦌`) where possible `StandardSimplex.mk n` is replaced with `⦋n⦌` where possible (except in notation and macros, which are left untouched). This includes opening `Simplicial` in two files. Also, outdated and unused `local notation` `[n]` for `StandardSimplex.mk n` is removed. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology 38/39 Mathlib/AlgebraicTopology/CechNerve.lean,Mathlib/AlgebraicTopology/MooreComplex.lean,Mathlib/AlgebraicTopology/SimplexCategory/Basic.lean,Mathlib/AlgebraicTopology/SimplicialObject/Basic.lean,Mathlib/AlgebraicTopology/SimplicialSet/Coskeletal.lean,Mathlib/AlgebraicTopology/SimplicialSet/NerveAdjunction.lean,Mathlib/AlgebraicTopology/SimplicialSet/StdSimplex.lean 7 1 ['github-actions'] nobody none
9-65931
9 days ago
9-76510
9 days ago
9-76563
9 days
25315 ocfnash
author:ocfnash
feat: add `simp` to lemma `Fin.coe_ofNat_eq_mod` One consequence is that `simp` can now prove things like this: ```lean example : (3 : Fin 10).val = 3 := by simp example : (4 : Fin 10).val = 4 := by simp example : (5 : Fin 10).val = 5 := by simp ``` previously this only this only worked up to `(2 : Fin 10).val = 2` (via lemmas like `Fin.val_two`). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data 32/28 Archive/Imo/Imo2024Q5.lean,Mathlib/AlgebraicTopology/DoldKan/Faces.lean,Mathlib/Analysis/CStarAlgebra/SpecialFunctions/PosPart.lean,Mathlib/Data/Fin/Basic.lean,Mathlib/Data/Fin/Parity.lean,Mathlib/Data/Fin/Rev.lean,Mathlib/GroupTheory/CommutingProbability.lean,Mathlib/GroupTheory/Perm/Fin.lean,Mathlib/RingTheory/ChainOfDivisors.lean,MathlibTest/matrix.lean 10 25 ['b-mehta', 'eric-wieser', 'github-actions', 'leanprover-bot', 'mattrobball', 'ocfnash'] nobody 1
9-18565
9 days ago
10-11743
10 days ago
10-11733
10 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 9 ['YaelDillies', 'erdOne', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant'] nobody none
9-11474
9 days ago
9-11493
9 days ago
12-10225
12 days
25284 alreadydone
author:alreadydone
feat(LinearAlgebra/Contraction): bijectivity of `dualTensorHom` + generalize to CommSemiring --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
168/44 Mathlib/Data/Finsupp/Defs.lean,Mathlib/LinearAlgebra/Contraction.lean,Mathlib/LinearAlgebra/Pi.lean,Mathlib/LinearAlgebra/Trace.lean,Mathlib/RingTheory/Finiteness/Finsupp.lean 5 5 ['alreadydone', 'eric-wieser', 'github-actions', 'leanprover-bot'] nobody none
8-77320
8 days ago
11-79692
11 days ago
11-79677
11 days
25078 loefflerd
author:loefflerd
feat(NumberTheory/ModularForms): GL(2, R) action preserves holomorphy Show that the slash action of negative-determinant matrices preserves holomorphic functions. --- - [x] depends on: #25028 - [x] depends on: #24740 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-number-theory 58/19 Mathlib/Analysis/Complex/UpperHalfPlane/Manifold.lean,Mathlib/NumberTheory/ModularForms/Basic.lean 2 5 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody none
8-38192
8 days ago
11-30057
11 days ago
11-30259
11 days
25343 plp127
author:plp127
docs(Topology/Perfect): Mention dense-in-itself The file `Mathlib/Topology/Perfect` defines a "nonstandard" predicate `Preperfect C` to mean that every point of `C` is an accumulation point of `C`. This property already has a name, it is called [dense-in-itself](https://en.wikipedia.org/wiki/Dense-in-itself). This PR adds this name to the docs. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology documentation 7/7 Mathlib/Topology/Perfect.lean 1 1 ['github-actions'] nobody none
8-27307
8 days ago
8-27385
8 days ago
8-27370
8 days
24777 joelriou
author:joelriou
feat(CategoryTheory): abstract argument for the stability under transfinite compositions If a class of morphisms is multiplicative, respects isomorphisms and is stable under filtered colimits, then it is stable under transfinite compositions. (This simplifies the proof in the case of monomorphisms in Grothendieck abelian categories, for isomorphisms, and in #23282, we shall apply this to monomorphisms in `Type`.) --- - [x] depends on: #24773 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-category-theory 122/116 Mathlib/CategoryTheory/Abelian/GrothendieckAxioms/Colim.lean,Mathlib/CategoryTheory/Abelian/GrothendieckCategory/EnoughInjectives.lean,Mathlib/CategoryTheory/Abelian/GrothendieckCategory/Monomorphisms.lean,Mathlib/CategoryTheory/MorphismProperty/Limits.lean,Mathlib/CategoryTheory/MorphismProperty/TransfiniteComposition.lean 5 12 ['callesonne', 'github-actions', 'joelriou', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody 1
8-11882
8 days ago
9-4698
9 days ago
21-28102
21 days
24514 b-mehta
author:b-mehta
chore(Int/GCD): use fuel in xgcd Modify the definition of xgcd to use fuel recursion, to allow it to be reduced in the kernel. As a consequence, this means the evaluation of field operations in ZMod p become provable by `rfl` and `decide`. Zulip discussion: https://leanprover.zulipchat.com/#narrow/channel/270676-lean4/topic/opaque.20recursion.20definitions.20break.20mergeSort.20decidability --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data 44/22 Mathlib/Data/Int/GCD.lean 1 4 ['b-mehta', 'eric-wieser', 'github-actions', 'nomeata', 'urkud'] nobody 1
7-84218
7 days ago
39-19437
1 month ago
39-19489
39 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 none
7-62144
7 days ago
8-71866
8 days ago
8-71857
8 days
24320 robin-carlier
author:robin-carlier
chore(Category/Theory/Whiskering): tag `[reassoc]` some lemmas about isoWhisker Using the extension of `reassoc` to equality of isomorphisms, tags some lemmas in `CategoryTheory.Whiskering` with this new version of the attribute. --- - [ ] depends on: #24303 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory 179/11 Mathlib.lean,Mathlib/CategoryTheory/Whiskering.lean,Mathlib/Tactic.lean,Mathlib/Tactic/CategoryTheory/IsoReassoc.lean,Mathlib/Tactic/CategoryTheory/Reassoc.lean,MathlibTest/CategoryTheory/Reassoc.lean 6 5 ['github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'robin-carlier'] nobody none
7-47673
7 days ago
7-47694
7 days ago
7-52796
7 days
25327 YaelDillies
author:YaelDillies
feat: `F.obj M` is a commutative monoid object if `M` is From Toric --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) toric 11/3 Mathlib/CategoryTheory/Monoidal/CommMon_.lean,Mathlib/CategoryTheory/Monoidal/Mon_.lean 2 1 ['github-actions'] nobody none
7-35334
7 days ago
9-34472
9 days ago
9-34465
9 days
25358 YaelDillies
author:YaelDillies
chore: more shortcut instances for `ℤ` Currently, some of those instances are inferred from `Int.instNormedCommRing : NormedCommRing ℤ` once one imports `Mathlib.Analysis.Normed.Ring.Lemmas`. Among other things, this confuses `#min_imports`, which then invariably reports that `Mathlib.Analysis.Normed.Ring.Lemmas` is used. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra easy
label:t-algebra$
16/5 Mathlib/Algebra/Ring/Int/Defs.lean,Mathlib/NumberTheory/LegendreSymbol/GaussEisensteinLemmas.lean,Mathlib/NumberTheory/Zsqrtd/QuadraticReciprocity.lean 3 4 ['eric-wieser', 'github-actions', 'leanprover-bot'] nobody none
7-29639
7 days ago
7-38392
7 days ago
7-39164
7 days
25186 riccardobrasca
author:riccardobrasca
feat: add `isPrincipalIdealRing_of_isPrincipal_of_lt_or_isPrincipal_of_mem_primesOver_of_mem_Icc` The standard technique to prove that `𝓞 K` is principal in the Galois case. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-number-theory 45/9 Mathlib/NumberTheory/NumberField/ClassNumber.lean 1 14 ['faenuccio', 'github-actions', 'riccardobrasca'] nobody none
6-37000
6 days ago
15-29033
15 days ago
15-29036
15 days
25235 ADedecker
author:ADedecker
feat: unit space of a (locally) compact T1 monoid is (locally) compact --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-topology 50/0 Mathlib/Topology/Algebra/Constructions.lean,Mathlib/Topology/Algebra/Group/Basic.lean 2 2 ['ADedecker', 'github-actions'] nobody none
6-24085
6 days ago
13-30528
13 days ago
13-30513
13 days
24884 smmercuri
author:smmercuri
feat: `ramificationIdx` for `NumberField.InfinitePlace` --- - [x] depends on: #24880 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-number-theory 38/0 Mathlib/NumberTheory/NumberField/InfinitePlace/Ramification.lean 1 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'riccardobrasca'] nobody none
6-19398
6 days ago
21-24116
21 days ago
21-24464
21 days
24875 smmercuri
author:smmercuri
feat: injectivity of `InfinitePlace.embedding` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-number-theory 19/0 Mathlib/NumberTheory/NumberField/InfinitePlace/Basic.lean 1 6 ['Ruben-VandeVelde', 'github-actions', 'riccardobrasca', 'smmercuri', 'xroblot'] nobody none
5-34998
5 days ago
26-48588
26 days ago
26-48642
26 days
25259 Thmoas-Guan
author:Thmoas-Guan
feat(Algebra): associated primes of localized module We proved the `Ass(S^{-1}M)` is equal to the preimage of `Ass(M)` under `Ideal.comap` when over noetherian ring. From this we proved that every minimal primes 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$
70/11 Mathlib/RingTheory/Ideal/AssociatedPrime/Localization.lean 1 6 ['Thmoas-Guan', 'erdOne', 'github-actions', 'leanprover-community-bot-assistant'] nobody none
4-53977
4 days ago
11-30057
11 days ago
12-23956
12 days
25172 eric-wieser
author:eric-wieser
feat: restricting `Affine.Simplex` to an affine subspace that contains it Also removes a redundant `Nonempty` argument. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) maintainer-merge t-euclidean-geometry 68/5 Mathlib/LinearAlgebra/AffineSpace/AffineSubspace/Basic.lean,Mathlib/LinearAlgebra/AffineSpace/Independent.lean 2 10 ['eric-wieser', 'github-actions', 'jsm28', 'ocfnash'] nobody 1
4-16192
4 days ago
15-26171
15 days ago
15-67045
15 days
25030 Multramate
author:Multramate
feat(NumberTheory/EllipticDivisibilitySequence): add elliptic nets Defines elliptic nets and redefines elliptic sequences using elliptic relators. This is part of #13057 by Junyan Xu. Co-authored-by: Junyan Xu --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-number-theory 259/37 Mathlib/NumberTheory/EllipticDivisibilitySequence.lean 1 1 ['github-actions'] nobody none
3-33209
3 days ago
17-77730
17 days ago
17-77714
17 days
25215 mans0954
author:mans0954
feature(RingTheory/RootsOfUnity/Basic) : rootsOfUnity coercions For a commutative monoid, `rootsOfUnity` can be coerced to the set `{z : R | z^k = 1}`. For a commutative ring which is a domain, `rootsOfUnity` can be coerced to `nthRootsFinset k (1 : R)`. Zulip discussion: https://leanprover.zulipchat.com/#narrow/channel/116395-maths/topic/roots.20of.20unity.20-.20computing.20low.20degree/with/520362922 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
22/0 Mathlib/RingTheory/RootsOfUnity/Basic.lean 1 1 ['github-actions'] nobody none
2-39154
2 days ago
14-10564
14 days ago
14-10619
14 days
24828 mans0954
author:mans0954
feature(Algebra/Polynomial/Roots) : nthRoots_two_unit_of_char_ne_two Compute the second roots of the unit for rings of characteristic not 2. See also: #25215 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
11/0 Mathlib/Algebra/Polynomial/Roots.lean,Mathlib/Data/Multiset/ZeroCons.lean 2 1 ['github-actions'] nobody none
2-39084
2 days ago
27-53731
27 days ago
27-59865
27 days
24809 robin-carlier
author:robin-carlier
feat(CategoryTheory/Functor/KanExtension): preservations of Kan extensions Introduce a typeclass `G.PreservesLeftKanExtension F L` that asserts that a functor `G` preserves the left Kan extension of `F` along a functor `L`. Introduce a pointwise variant, and relate it to the non-pointwise version when pointwise extensions exist. Show that a functor that preserves the relevant colimits preserve pointwise left Kan extensions. Construct isomorphisms `L.leftKanExtension F ⋙ G ≅ L.leftKanExtension (F ⋙ G)` when `G.PreservesLeftKanExtension F L` holds. Also construct a functorial version, as an isomorphism `L.lan ⋙ (whiskeringRight _ _ _).obj G ≅ (whiskeringRight _ _ _).obj G ⋙ L.lan`. All results are dualised to right Kan extensions. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory 551/0 Mathlib.lean,Mathlib/CategoryTheory/Functor/KanExtension/Basic.lean,Mathlib/CategoryTheory/Functor/KanExtension/Preserves.lean 3 5 ['TwoFX', 'github-actions', 'joelriou', 'robin-carlier'] nobody none
2-25051
2 days ago
28-28334
28 days ago
28-28383
28 days
25331 fbarroero
author:fbarroero
feat(RingTheory/Ideal/Maximal): `ne_top_iff_exists_maximal` We add `Ideal.ne_top_iff_exists_maximal` and an analogous statement for `IsDedekindDomain.HeightOneSpectrum`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
18/0 Mathlib/RingTheory/DedekindDomain/Ideal.lean,Mathlib/RingTheory/Ideal/Maximal.lean 2 5 ['Ruben-VandeVelde', 'fbarroero', 'github-actions'] nobody none
2-7027
2 days ago
9-18489
9 days ago
9-18541
9 days
25174 zcyemi
author:zcyemi
feat(Geometry/Euclidean/Triangle): add law of sines --- Implement the vector and angle-at-point forms of the law of sines. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-euclidean-geometry 57/1 Mathlib/Geometry/Euclidean/Triangle.lean 1 15 ['eric-wieser', 'github-actions', 'jsm28', 'zcyemi'] nobody none
1-29741
1 day ago
15-50897
15 days ago
15-50951
15 days
22834 joelriou
author:joelriou
feat(CategoryTheory): lifting properties and parametrized adjunctions Given a parametrized adjunction `adj₂ : F ⊣₂ G` between bifunctors `F : C₁ ⥤ C₂ ⥤ C₃` and `G : C₁ᵒᵖ ⥤ C₃ ⥤ C₂`, three maps `f₁ : X₁ ⟶ Y₁` in `C₁`, `f₂ : X₂ ⟶ Y₂` in `C₂`, and `f₃ : X₃ ⟶ Y₃` in `C₃`, this PR shows that `f₃` has the right lifting property with respect to the "inclusion" of the pushout of `(F.obj Y₁).obj X₂` and `(F.obj X₁).obj Y₂` along `(F.obj X₁).obj X₂` into `(F.obj Y₁).obj Y₂` if and only if `f₂` has the left lifting property with respect to the projection map from `(G.obj Y₁).obj X₃` to the pullback of `(G.obj (op X₁)).obj X₃` and `(G.obj (op Y₁)).obj Y₃` over `(G.obj (op X₁)).obj Y₃`. (In homotopical algebra, this is typically used for the adjunction between the tensor product and the internal hom.) --- - [x] depends on: #22828 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory 309/0 Mathlib.lean,Mathlib/CategoryTheory/LiftingProperties/Basic.lean,Mathlib/CategoryTheory/LiftingProperties/ParametrizedAdjunction.lean 3 10 ['github-actions', 'joelriou', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'robin-carlier'] nobody none
1-9993
1 day ago
17-77605
17 days ago*
17-77596
17 days*
25348 wwylele
author:wwylele
feat(LinearAlgebra): add independent iSup to LinearPMap This is part of #25140. To obtain the Hahn embedding, we need to construct an partial linear map spanned by a family of submodules as the base case. This PR prepares for it. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-algebra
label:t-algebra$
94/2 Mathlib/LinearAlgebra/DFinsupp.lean,Mathlib/LinearAlgebra/LinearPMap.lean 2 2 ['eric-wieser', 'github-actions'] nobody none
0-72911
20 hours ago
8-9468
8 days ago
8-9532
8 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$
92/1 Mathlib.lean,Mathlib/Algebra/Ring/Equiv.lean,Mathlib/RingTheory/RingHom/FaithfullyFlat.lean,Mathlib/RingTheory/RingHom/Flat.lean 4 4 ['chrisflav', 'erdOne', 'github-actions', 'mathlib4-dependent-issues-bot'] nobody 1
0-42212
11 hours ago
30-36220
30 days ago
30-37286
30 days
13611 callesonne
author:callesonne
feat(FiberedCategory/HasFibers): define HasFibers class We define a class `HasFibers p` for a given functor `p : 𝒳 ⥤ 𝒮`. The point of this is to give the user the option to supply their own fiber categories, as often the standard fibers will not be definitionally the same as the (equivalent) categories one is interested in. Co-authored-by: Paul Lezeau --- This is the final PR in a sequence of PRs developing the theory of fibered categories that I will make for now. I will wait for the reviewing to catch up before I start working on more of these again, so as to not create too big of a backlog. - [x] depends on: #13603 - [x] depends on: #12982 - [x] depends on: #13416 - [x] depends on: #13410 - [x] depends on: #13393 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory 276/21 Mathlib.lean,Mathlib/CategoryTheory/FiberedCategory/Cartesian.lean,Mathlib/CategoryTheory/FiberedCategory/HasFibers.lean,Mathlib/CategoryTheory/FiberedCategory/HomLift.lean 4 26 ['callesonne', 'github-actions', 'joelriou', 'mathlib4-dependent-issues-bot'] nobody none
0-40081
11 hours ago
233-21757
7 months ago*
0-571
9 minutes*
24379 chrisflav
author:chrisflav
feat(Algebra/AlgHom): `Unique` if target is `Subsingleton` --- [![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/Algebra/Equiv.lean,Mathlib/Algebra/Algebra/Hom.lean 2 6 ['chrisflav', 'eric-wieser', 'github-actions'] nobody none
0-38535
10 hours ago
39-28735
1 month ago
39-64672
39 days
25334 matthewjasper
author:matthewjasper
feat(RingTheory/Flat): Add theorems relating Submodule.torsion and Module.Flat Co-authored-by: Kevin Buzzard --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) FLT new-contributor t-algebra
label:t-algebra$
202/0 Mathlib.lean,Mathlib/Algebra/Algebra/Bilinear.lean,Mathlib/Algebra/Module/LocalizedModule/Basic.lean,Mathlib/RingTheory/Flat/TorsionFree.lean,Mathlib/RingTheory/Ideal/IsPrincipal.lean 5 13 ['alreadydone', 'erdOne', 'github-actions', 'kbuzzard'] nobody none
0-24330
6 hours ago
9-7627
9 days ago
9-7626
9 days
25365 YaelDillies
author:YaelDillies
feat: `CommAlgCat` is cocartesian-monoidal Construct the cocartesian-monoidal category structure on `CommAlgCat R` explicitly from the tensor product. From Toric Co-authored-by: Andrew Yang Co-authored-by: Michał Mrugała Co-authored-by: Christian Merten --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) toric t-algebra
label:t-algebra$
142/5 Mathlib.lean,Mathlib/Algebra/Category/CommAlgCat/Basic.lean,Mathlib/Algebra/Category/CommAlgCat/Monoidal.lean 3 8 ['YaelDillies', 'erdOne', 'github-actions'] nobody none
0-18718
5 hours ago
7-26981
7 days ago
7-28134
7 days
25168 wwylele
author:wwylele
feat(RingTheorey/HahnSeries): equip HahnSeries with LinearOrder This is part of #25140. As the future codomain of Hahn embedding theorem, `HahnSeries` needs a linear order. ~~It might be debatable whether the lexicographical order should be *the* order of `HahnSeries`. Aside from usage in Hahn embedding theorem, this order also represents, for example, the asymptotic behavior around `(x : R) = 0`, so it is generally useful.~~ Updated to add `LinearOrder` on `Lex (HahnSeries _ _)` instead --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
180/0 Mathlib.lean,Mathlib/RingTheory/HahnSeries/Addition.lean,Mathlib/RingTheory/HahnSeries/Basic.lean,Mathlib/RingTheory/HahnSeries/Lex.lean 4 10 ['ScottCarnahan', 'eric-wieser', 'github-actions', 'wwylele'] nobody none
0-5576
1 hour ago
15-72780
15 days ago
15-72831
15 days

Stale assigned PRs on the review queue

Number Author Title Description Labels +/- Modified files (first 100) 📝 💬 All users who commented or reviewed Assignee(s) Approval(s) Updated Last status change total time in review
20719 gio256
author:gio256
feat(AlgebraicTopology): delaborators for truncated simplicial notations We add delaborators for the following notations, introduced in #20688: - `⦋m⦌ₙ`, which denotes the `m`-dimensional simplex in the `n`-truncated simplex category. - `X _⦋m⦌ₙ`, which denotes the `m`-th term of an `n`-truncated simplicial object `X`. - `X ^⦋m⦌ₙ`, which denotes the `m`-th term of an `n`-truncated cosimplicial object `X`. If `pp.proofs` is set to `true`, we also pretty-print the proof `p : m ≤ n` for all three notations as `⦋m, p⦌ₙ`, `X _⦋m, p⦌ₙ`, and `X ^⦋m, p⦌ₙ`, respectively. Credit to @kmill for one piece of code and much metaprogramming inspiration. --- - [x] depends on: #20688 - [x] depends on: #23018 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) infinity-cosmos t-category-theory t-meta 525/33 Mathlib.lean,Mathlib/AlgebraicTopology/SimplexCategory/Basic.lean,Mathlib/AlgebraicTopology/SimplexCategory/Defs.lean,Mathlib/AlgebraicTopology/SimplicialObject/Basic.lean,Mathlib/Tactic.lean,Mathlib/Tactic/SimplexCategory.lean,Mathlib/Util/Superscript.lean,MathlibTest/SimplexCategory.lean,MathlibTest/SimplicialObject.lean,MathlibTest/superscript.lean,scripts/noshake.json 11 22 ['eric-wieser', 'gio256', 'github-actions', 'kim-em', 'mathlib4-dependent-issues-bot'] eric-wieser
assignee:eric-wieser
none
39-7178
1 month ago
39-9819
1 month ago
47-81361
47 days
22464 adomani
author:adomani
feat(CI): declarations diff in Lean Rewrites the `declaration_diff` script in Lean. You can see the effect of the new script in the testing branch #22497. The new CI step runs in approximately 5mins, but is separate from the `build` step. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) CI 151/0 .github/workflows/PR_summary_lean.yml,scripts/README.md,scripts/declarations_diff.lean,scripts/declarations_diff_lean_shell_glue.sh 4 6 ['bryangingechen', 'github-actions', 'grunweg'] robertylewis
assignee:robertylewis
none
32-46758
1 month ago
97-11003
3 months ago
97-10992
97 days
24172 LessnessRandomness
author:LessnessRandomness
feat: specialize rational root theorem to usual rational numbers and integers Rational root theorem and integral root theorem - the special case for usual rational numbers and integers. --- new-contributor t-algebra
label:t-algebra$
123/0 Mathlib.lean,Mathlib/RingTheory/Polynomial/OfRationalNumbers/RationalRootTheorem.lean 2 2 ['github-actions', 'grunweg'] mariainesdff
assignee:mariainesdff
none
32-46491
1 month ago
52-14174
1 month ago
52-14228
52 days
22792 madvorak
author:madvorak
feat(Mathlib/Data/Fin/Pigeonhole): pigeonhole-like results for Fin Consider the following settings: ``` import Mathlib example (X Y : Type) [Fintype X] [Fintype Y] (f : X → Y) (hf : f.Injective) : Fintype.card X ≤ Fintype.card Y := by hint example (m n : ℕ) (f : Fin m → Fin n) (hf : f.Injective) : m ≤ n := by hint example (X Y : Type) [Fintype X] [Fintype Y] (f : X ↪ Y) : Fintype.card X ≤ Fintype.card Y := by hint example (m n : ℕ) (f : Fin m ↪ Fin n) : m ≤ n := by hint ``` The 1st and 3rd `hint` succeed, but the 2nd a 4th `hint` fail. The problem is obviously that `exact?` does not see through `Fintype.card (Fin n) = n` when searching for appropriate lemma. It may seem to not be a problem, as it will rarely derail experienced Mathlib users — after all, experienced Leaners usually go directly for the `Finset` or `Fintype` version. However, beginners frequently work with `Fin` and they will expect stuff like ``` theorem le_of_injective (f : Fin m → Fin n) (hf : f.Injective) : m ≤ n ``` to exist; therefore, when `hint` or `exact?` fails, it is a very unpleasant surprise. This PR addressed this issue; not to provide useful content for advanced users, but to make Mathlib more useful for beginners. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data 38/0 Mathlib.lean,Mathlib/Data/Fin/Pigeonhole.lean 2 1 ['github-actions'] ericrbg
assignee:ericrbg
none
32-26308
1 month ago
91-16059
2 months ago
91-16110
91 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
none
32-26230
1 month ago
52-85074
1 month ago
63-47491
63 days
23826 javra
author:javra
feat(CategoryTheory): linear categories as `ModuleCat R`-enriched categories --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-category-theory 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 2 ['github-actions', 'leanprover-community-bot-assistant'] TwoFX
assignee:TwoFX
none
32-26214
1 month ago
56-36648
1 month ago
56-36630
56 days
24054 plp127
author:plp127
feat(Topology): R1 spaces are quasisober This generalizes `T2Space.quasiSober` --- - [ ] depends on: #24098 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology 36/8 Mathlib/Topology/Separation/Basic.lean,Mathlib/Topology/Separation/Hausdorff.lean,Mathlib/Topology/Sober.lean 3 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'urkud'] urkud
assignee:urkud
none
32-19721
1 month ago
47-9884
1 month ago
48-19934
48 days
23678 plp127
author:plp127
feat: recursor for nonempty lists Adds `List.recNeNil` and `List.recOnNeNil` for motives that depend on the list being nonempty. Taken from [Zulip](https://leanprover.zulipchat.com/#narrow/channel/217875-Is-there-code-for-X.3F/topic/accessing.20the.20source.20case.20during.20induction/near/502101211). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data 40/0 Mathlib/Data/List/Induction.lean 1 6 ['eric-wieser', 'github-actions', 'plp127'] ericrbg
assignee:ericrbg
none
31-75873
1 month ago
66-2110
2 months ago
66-2161
66 days
23930 Vtec234
author:Vtec234
feat(Tactic): dependent rewriting 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 --- 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 706/0 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/DepRewrite.lean,MathlibTest/depRewrite.lean 4 1 ['github-actions'] adamtopaz
assignee:adamtopaz
none
31-75742
1 month ago
59-70313
1 month ago
59-70362
59 days
22196 xyzw12345
author:xyzw12345
feat: `lie_ring` tactic and `LieReduce` command In this PR, we implement a new tactic that reduces expressions in a `LieRing` to a normal form and checks whether they are equal, and a command which reduces the expression and displays the normal form. The implementation of this tactic imitates the `ring` tactic, using the `Qq` package to implement a specific reduction algorithm, following the theory of Hall sets and Lyndon words. A reference for the algorithm can be found at, for example, [here](https://personal.math.ubc.ca/~cass/research/pdf/Free.pdf). This project is the result of a workshop at Peking University, and @siddhartha-gadgil has helped us a lot on understanding the concepts in metaprogramming. Edit: The changes are reverted to a point where only `AtomM` is used. Co-authored-by: @Thmoas-Guan <2300010733@stu.pku.edu.cn> @yhtq <2100012990@stu.pku.edu.cn> @Blackfeather007 <2100017455@stu.pku.edu.cn> --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-meta 816/2 Mathlib.lean,Mathlib/Algebra/Lie/Derivation/AdjointAction.lean,Mathlib/Tactic.lean,Mathlib/Tactic/LieAlgebra/Basic.lean,Mathlib/Tactic/LieAlgebra/LieRingNF.lean,Mathlib/Util/AtomM.lean,MathlibTest/lie_ring.lean,scripts/noshake.json 8 16 ['bryangingechen', 'eric-wieser', 'faenuccio', 'github-actions', 'grunweg', 'ocfnash', 'siddhartha-gadgil', 'xyzw12345'] robertylewis
assignee:robertylewis
none
31-30093
1 month ago
106-61592
3 months ago
106-61583
106 days
24036 Louddy
author:Louddy
feat: add `HeightOneSpectrum.ofPrime` Add a definition relating elements of type `HeightOneSpectrum R` with the (nonzero) prime elements of the monoid with zero `Ideal R`. (Note the distinction between `Prime` and `Ideal.IsPrime`). The documentation string is inspired from [Ideal.prime_iff_isPrime](https://leanprover-community.github.io/mathlib4_docs/Mathlib/RingTheory/DedekindDomain/Ideal.html#Ideal.prime_iff_isPrime). This was discussed [#mathlib4 > Placing a definition in `DedekindDomain.Ideal` @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Placing.20a.20definition.20in.20.60DedekindDomain.2EIdeal.60/near/511647129). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra
label:t-algebra$
11/1 Mathlib/RingTheory/DedekindDomain/Ideal.lean 1 5 ['Louddy', 'Ruben-VandeVelde', 'github-actions'] Ruben-VandeVelde
assignee:Ruben-VandeVelde
1
31-28220
1 month ago
56-29490
1 month ago
56-29544
56 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 27 ['YaelDillies', 'b-mehta', 'eric-wieser', 'github-actions', 'kbuzzard', 'kmill', 'leanprover-community-mathlib4-bot'] kmill
assignee:kmill
none
31-28133
1 month ago
78-2807
2 months ago
126-22495
126 days
22089 sgouezel
author:sgouezel
feat: composing a continuous multilinear map with continuous linear maps is analytic in both variables Also prove that the composition of continuously polynomial functions is continuously polynomial. --- - [x] depends on: #22102 - [x] depends on: #22789 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis 277/80 Mathlib/Analysis/Analytic/CPolynomial.lean,Mathlib/Analysis/Analytic/Composition.lean,Mathlib/Analysis/NormedSpace/Multilinear/Basic.lean,Mathlib/Data/Multiset/DershowitzManna.lean,Mathlib/Order/KrullDimension.lean 5 9 ['github-actions', 'grunweg', 'mathlib4-dependent-issues-bot', 'sgouezel', 'urkud'] loefflerd
assignee:loefflerd
none
31-23140
1 month ago
69-4593
2 months ago
107-57540
107 days
23320 Whysoserioushah
author:Whysoserioushah
feat(Mathlib/RingTheory/TwoSidedIdeal/SpanAsSum): span of set as finsum co-authored by: @jjaassoonn --- splited from [#23216](https://github.com/leanprover-community/mathlib4/pull/23216) following @eric-wieser advice [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
81/0 Mathlib.lean,Mathlib/RingTheory/TwoSidedIdeal/SpanAsSum.lean 2 43 ['Paul-Lez', 'Whysoserioushah', 'eric-wieser', 'github-actions', 'kbuzzard'] eric-wieser
assignee:eric-wieser
none
31-21018
1 month ago
75-73462
2 months ago
75-73506
75 days
23459 Timeroot
author:Timeroot
feat: Definition of `Clone` notations and typeclasses Definitions and notation typeclasses for #20051 --- [![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/Clone/Defs.lean 2 22 ['Timeroot', 'YaelDillies', 'dupuisf', 'eric-wieser', 'github-actions', 'urkud'] YaelDillies
assignee:YaelDillies
none
30-81075
30 days ago
63-17358
2 months ago
65-66460
65 days
17627 hrmacbeth
author:hrmacbeth
feat: universal properties of vector bundle constructions Characterizations for the smoothness of maps into the total spaces of (1) the direct sum of two vector bundles; (2) the pullback of a vector bundle. This gap in the library was exposed by #17358. --- - [x] depends on: #22804 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-differential-geometry 311/9 Mathlib/Data/Bundle.lean,Mathlib/Geometry/Manifold/VectorBundle/Basic.lean,Mathlib/Geometry/Manifold/VectorBundle/Pullback.lean,Mathlib/Topology/FiberBundle/Constructions.lean 4 14 ['github-actions', 'grunweg', 'hrmacbeth', 'j-loreaux', 'mathlib4-dependent-issues-bot', 'sgouezel'] grunweg
assignee:grunweg
none
27-82562
27 days ago
81-30618
2 months ago
82-15074
82 days
24372 Hagb
author:Hagb
feat(Tactic/SimpIntro): add support for introducing non-propositions `simp_intro` would be able to introduce non-propositions. The previous `simp_intro` tactic cannot solve some statement that can be solved by applying `intro` and `simp` like `simp_intro`. For example, the following one can be solved like this ```lean example (r : Nat → Prop) : (∀ x, x > 0 → r x) → ∀ y z, y = 0 → z > y → r z := by simp intro hr try simp at hr -- does nothing try simp [hr] -- does nothing intro y z try simp [hr] -- does nothing intro hy try simp [hr] at hy -- does nothing simp [hr, hy] intro hyz try simp [hr, hy] at hyz simp [hr, hy, hyz] -- accomplish the goal successfully ``` while the previous `simp_intro` cannot introduce `y` and `z` here. ```lean example (r : Nat → Prop) : (∀ x, x > 0 → r x) → ∀ y z, y = 0 → z > y → r z := by /- the previous `simp_intro` fails with message: invalid 'simp', proposition expected Nat -/ simp_intro .. -- or `simp_intro hr y` example (r : Nat → Prop) : (∀ x, x > 0 → r x) → ∀ y z, y = 0 → z > y → r z := by -- unsolved simp_intro hr example (r : Nat → Prop) : (∀ x, x > 0 → r x) → ∀ y z, y = 0 → z > y → r z := by -- successfully solve the goal with the `simp_intro` in thie commit simp_intro .. -- or `simp_intro hr y z hy hz` ``` This commit makes it be able to introduce these kinds of hypotheses. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-meta 13/2 Mathlib/Tactic/SimpIntro.lean,MathlibTest/simp_intro.lean 2 1 ['github-actions'] kmill
assignee:kmill
none
27-81860
27 days ago
45-5392
1 month ago
45-5443
45 days
24395 rudynicolop
author:rudynicolop
feat(Data/List): list splitting definitions and lemmas Adds definitions and lemmas for obtaining all prefixes and suffixes of lists. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data new-contributor 143/2 Mathlib/Data/List/Perm/Lattice.lean,Mathlib/Data/List/TakeDrop.lean 2 1 ['github-actions'] ericrbg
assignee:ericrbg
none
27-81842
27 days ago
44-2869
1 month ago
44-2931
44 days
23955 Louddy
author:Louddy
feat: Ideal.count_associates_eq Add variant of `UniqueFactorizationMonoid.count_normalizedFactors_eq` for associated Ideals. This is convenient when you need to talk about an element as `a₀ = x ^ n * a`. Note the file is slightly over the 1500 lines limit, I hope that is ok. 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/) new-contributor t-algebra
label:t-algebra$
35/1 Mathlib/RingTheory/DedekindDomain/Ideal.lean 1 7 ['Louddy', 'Ruben-VandeVelde', 'alreadydone', 'github-actions', 'grunweg'] kbuzzard
assignee:kbuzzard
1
26-44624
26 days ago
26-44624
26 days ago
53-45384
53 days
19796 peakpoint
author:peakpoint
feat: L'Hopital's rule from within a convex set --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-analysis 190/19 Mathlib/Algebra/Polynomial/Module/Basic.lean,Mathlib/Analysis/Calculus/LHopital.lean,Mathlib/Analysis/Convex/Topology.lean,Mathlib/Geometry/Manifold/Instances/Real.lean,Mathlib/Order/Interval/Set/Basic.lean 5 14 ['RemyDegenne', 'github-actions', 'leanprover-community-bot-assistant', 'peakpoint', 'sgouezel'] sgouezel
assignee:sgouezel
none
21-79134
21 days ago
21-79134
21 days ago
55-29418
55 days
20240 mitchell-horner
author:mitchell-horner
feat(Combinatorics/SimpleGraph): prove the Kővári–Sós–Turán theorem Prove the Kővári–Sós–Turán theorem for simple graphs: the `(completeBipartiteGraph α β).Free` simple graphs for `card α ≤ card β` on the vertex type `V` have at most `(card β-1)^(1/(card α))*(card V)^(2-1/(card α))/2 + (card V)*(card α-1)/2` edges. --- - [x] depends on: #19865 - [x] depends on: #20738 I'd like to make `aux` not private in the `KovariSosTuran` namespace to enable reuse of the double-counting here, but I don't know what to call it. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-combinatorics 289/0 Mathlib.lean,Mathlib/Combinatorics/SimpleGraph/Bipartite.lean,Mathlib/Combinatorics/SimpleGraph/Extremal/KovariSosTuran.lean 3 3 ['github-actions', 'mathlib4-dependent-issues-bot'] awainverse
assignee:awainverse
none
19-29414
19 days ago
41-69299
1 month ago
41-69833
41 days
22018 maddycrim
author:maddycrim
feat(RingTheory/Localization/Pi): localization of a finite direct product where each semiring in product has maximal nilradical is a projection For noncomputable def `surjectivePiNilradicalIsMaximal` : Let `M` be a submonoid of a direct product of commutative rings `R i`. If each `R i` has maximal nilradical then the direct product `∏ R i` surjects onto the localization of `∏ R i` at `M`. --- [![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$
28/0 Mathlib/RingTheory/Localization/Pi.lean 1 24 ['Paul-Lez', 'alreadydone', 'erdOne', 'github-actions', 'grunweg', 'jcommelin', 'maddycrim'] mariainesdff
assignee:mariainesdff
1
19-29279
19 days ago
64-12686
2 months ago
110-85911
110 days
22961 xroblot
author:xroblot
feat(ZLattice/Covolume): add `covolume_div_covolume_eq_relindex` Add the following result: Let `L₁` be a sub-`ℤ`-lattice of `L₂`. Then the index of `L₁` inside `L₂` is equal to `covolume L₁ / covolume L₂`. --- - [x] depends on: #22940 - [x] depends on: #23759 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
66/4 Mathlib/Algebra/Module/ZLattice/Basic.lean,Mathlib/Algebra/Module/ZLattice/Covolume.lean,Mathlib/GroupTheory/Index.lean,Mathlib/LinearAlgebra/Determinant.lean 4 10 ['Ruben-VandeVelde', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'xroblot'] ericrbg
assignee:ericrbg
none
19-29255
19 days ago
42-41084
1 month ago
78-83644
78 days
23681 Timeroot
author:Timeroot
feat(Algebra/Polynomial): Descartes' Rule of signs Proof of Descartes' Rule of Signs. Last PR from https://github.com/Timeroot/lean-descartes-signs , now that #9085 is merged. Defines `Polynomial.SignVariations` as the relevant quantity, and `descartes_rule_of_signs` as the headline theorem. --- I tried to clean it up + golf it down and did shrink it a good deal. The lemma `signvar_mul_eraseLead_le_of_nextCoeff` is still 142 lines, and `succ_sign_lin_mul` is ~140 lines of code as well. Those are the ugly ones. I welcome ideas if someone wants to try to clean them up more! But the proof really does require an annoying bit of case-splitting, as far as I can tell. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
615/3 Mathlib.lean,Mathlib/Algebra/Polynomial/CoeffList.lean,Mathlib/Algebra/Polynomial/Degree/Operations.lean,Mathlib/Algebra/Polynomial/EraseLead.lean,Mathlib/Algebra/Polynomial/RuleOfSigns.lean 5 6 ['BoltonBailey', 'Timeroot', 'github-actions', 'grunweg'] adomani
assignee:adomani
none
19-28937
19 days ago
65-82525
2 months ago
65-82572
65 days
23752 jsm28
author:jsm28
feat(Geometry/Euclidean/Incenter): incenters and excenters Define the exspheres and insphere of a simplex (in dimension 1 and greater), and corresponding definitions for their center and radius. Give necessary and sufficient conditions for them to exist (in terms of the barycentric coordinates, being signed versions of the inverses of the distances between vertices and opposite faces, having a nonzero sum) and show that they do always exist in the case of the incenter and of the excenter opposite a single vertex (the latter in dimensions 2 and greater), and that any point lying in the span of the vertices and equidistant from the faces opposite the vertices is an excenter (and, when signs of the equal distances are given, is the excenter with corresponding signs). Some major pieces are deferred to followups, in particular definitions of touchpoints, tangency of exspheres and insphere to faces, and the relation to angle bisectors in various forms. But since the file is already over 600 lines, I think this is a reasonable starting point (and since the lemmas do show that the definitions have their characteristic properties of points being equidistant from the faces on the desired sides, I think it sufficiently justifies that the definitions are correct and usable as-is). Feel free to golf; the calculations involved in showing that the excenter opposite a vertex always exists (in dimensions 2 and greater) are rather long. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) - [x] depends on: #23712 - [x] depends on: #23751 - [x] depends on: #24503 - [x] depends on: #24968 - [x] depends on: #25029 t-euclidean-geometry 556/0 Mathlib.lean,Mathlib/Data/Fin/Basic.lean,Mathlib/Geometry/Euclidean/Altitude.lean,Mathlib/Geometry/Euclidean/Incenter.lean 4 53 ['JovanGerb', 'eric-wieser', 'github-actions', 'jsm28', 'mathlib4-dependent-issues-bot'] eric-wieser
assignee:eric-wieser
none
19-26
19 days ago
20-11713
20 days ago
62-48480
62 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
none
18-68272
18 days ago
46-65829
1 month ago
46-65883
46 days
16074 Rida-Hamadani
author:Rida-Hamadani
feat: combinatorial maps and planar graphs We define combinatorial maps, then we define planar graph using combinatorial maps. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics 243/0 Mathlib.lean,Mathlib/Combinatorics/SimpleGraph/Planar.lean,Mathlib/Data/CombinatorialMap.lean 3 27 ['Parcly-Taxel', 'Rida-Hamadani', 'github-actions', 'lambda-fairy', 'leanprover-community-bot-assistant'] kmill
assignee:kmill
none
18-24212
18 days ago
43-35814
1 month ago
47-23245
47 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
none
18-24063
18 days ago
54-35449
1 month ago
109-82571
109 days
23926 b-reinke
author:b-reinke
feat(Algebra/BigOperators/Finprod): add powerset projection lemmas This PR adds lemmas in `Mathlib/Algebra/BigOperators/Finprod.lean` related to products/sums over the powerset `𝒫 s` when we add or remove an element of `s`. The motivation comes from the proof of the deletion/contraction properties of matroids. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
30/0 Mathlib/Algebra/BigOperators/Finprod.lean,Mathlib/Data/Set/Image.lean 2 5 ['b-reinke', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant'] joelriou
assignee:joelriou
none
18-23928
18 days ago
46-44557
1 month ago
59-45080
59 days
24139 yuanyi-350
author:yuanyi-350
feat: add `Fin.cycleIcc` which rotates `range(i, j)` In this file, I define permutation `cycleIcc i j hij`, which is the cycle `(i i+1 .... j)` leaving `(0 ... i-1)` and `(j+1 ... n-1)` unchanged. In other words, it rotates elements in `[i, j]` one step to the right. Also I prove some properties of `cycleIcc i j hij` such as it is a cycle and its cycleType is `j - i` **This definition is used to prove the following result:** ``` theorem succAbove_comp_cycleIcc [NeZero n] (x : Fin (n + 1) → L) (i j : Fin (n + 1)) (eq : x i = x j) (lt : i < j) x ∘ i.succAbove = x ∘ j.succAbove ∘ (cycleIcc hij) ``` More clearly, `x ∘ i.succAbove` and `x ∘ j.succAbove` are `Fin n → L` types. For example, when `n = 6, i = 2, j = 5` and `x i = x j` ``` x ∘ i.succAbove = (x 0, x 1, x 3, x 4, x 5, x 6) x ∘ j.succAbove = (x 0, x 1, x 2, x 3, x 4, x 6) ``` We have ``` (x 0, x 1, x 3, x 4, x 5, x 6) --(cycleIcc)--->(x 0, x 1, x 5, x 3, x 4, x 6) = (x 0, x 1, x 2, x 3, x 4, x 6) ``` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra
label:t-algebra$
132/1 Mathlib/Algebra/Group/Fin/Basic.lean,Mathlib/Data/Fin/Basic.lean,Mathlib/Data/Nat/SuccPred.lean,Mathlib/GroupTheory/Perm/Fin.lean 4 27 ['acmepjz', 'faenuccio', 'github-actions', 'grunweg', 'leanprover-bot', 'leanprover-community-bot-assistant', 'mbkybky', 'yuanyi-350'] faenuccio
assignee:faenuccio
none
18-23587
18 days ago
38-69996
1 month ago
52-84299
52 days
24546 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/) t-combinatorics 36/0 Mathlib/Combinatorics/SimpleGraph/Coloring.lean,Mathlib/Combinatorics/SimpleGraph/ConcreteColorings.lean,Mathlib/Combinatorics/SimpleGraph/Path.lean 3 3 ['IvanRenison', 'github-actions', 'jt496'] b-mehta
assignee:b-mehta
none
18-23441
18 days ago
38-24851
1 month ago
38-40361
38 days
21966 vasnesterov
author:vasnesterov
feat(Tactic/Order): support `⊤`, `⊥`, and lattice operations Support `⊤`, `⊥`, and lattice operations in the `order` tactic. --- - [x] depends on: #21877 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-meta 255/81 Mathlib/Tactic/Order.lean,Mathlib/Tactic/Order/CollectFacts.lean,Mathlib/Tactic/Order/Graph/Basic.lean,Mathlib/Tactic/Order/Preprocessing.lean,MathlibTest/order.lean,scripts/noshake.json 6 2 ['github-actions', 'mathlib4-dependent-issues-bot'] kmill
assignee:kmill
none
18-21038
18 days ago
67-38583
2 months ago
101-35078
101 days
24497 Parcly-Taxel
author:Parcly-Taxel
feat: IMO 1985 Q2 IMO 100/0 Archive.lean,Archive/Imo/Imo1985Q2.lean 2 1 ['github-actions'] dwrensha
assignee:dwrensha
none
16-10479
16 days ago
39-37793
1 month ago
39-37776
39 days
24517 upobir
author:upobir
feat(Algebra/QuadraticDiscriminant): Adding inequalities on quadratic from inequalities on discriminant --- This pr adds inequalities that relate `0` and `a * (x * x) + b * x + c` from inequalities of `a` and `discrim a b c`. For example, negative discriminant and negative leading coefficient implies value of quadratic expression is always negative and similar. [![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 1 ['github-actions'] chrisflav
assignee:chrisflav
none
16-10458
16 days ago
39-16657
1 month ago
39-16709
39 days
24522 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/) t-condensed 39/0 Mathlib.lean,Mathlib/Condensed/Light/Small.lean 2 1 ['github-actions'] joneugster
assignee:joneugster
none
16-10408
16 days ago
39-9950
1 month ago
39-10005
39 days
24685 robin-carlier
author:robin-carlier
feat(CategoryTheory/Limits/Preserves): Preservations of (co)limits by bifunctors Introduce a typeclass `PreservesColimit₂` that bundles the assumption that a bifunctor preserves a pair of colimit diagrams in each of its variables. This is stated in terms of a construction `Functor.mapCocone₂` that applies a bifunctor `G` to a pair of cocones to get a cocone over the uncurryfication of `whiskeringLeft₂ _|>.obj _|>.obj _|>.obj G`. The cocone points of this construction is definitionally the evaluation of `G` at the cocone points of the two cocones given as parameters. We give helper functions to extract isomorphisms with abstract colimits out of this typeclass, and we characterize these isomorphisms with respect to the canonical maps to the colimits. The dual typeclass for limits is also introduced. --- The definition of `Functor.mapCocone₂` and of `PreservesColimit₂` is due to @joelriou and was suggested during review of #17781. This PR only contains basic definitions, but does not give any interesting ways of inferring a `PreservesColimit₂` instance. This will be the content of a follow-up PR. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory 243/0 Mathlib.lean,Mathlib/CategoryTheory/Limits/Preserves/Bifunctor.lean 2 1 ['github-actions'] joelriou
assignee:joelriou
none
16-10290
16 days ago
32-15906
1 month ago
32-15960
32 days
24213 BoltonBailey
author:BoltonBailey
feat: add simp lemmas for trig functions on `π * 2⁻¹` This PR adds a number of simp lemmas to reduce trig functions evaluated on `π * 2⁻¹`. This allows `simp` to reduce expressions such as `sin (π * (1 / 2))` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis 45/0 Mathlib/Analysis/SpecialFunctions/Trigonometric/Basic.lean 1 3 ['YaelDillies', 'github-actions', 'leanprover-community-bot-assistant'] YaelDillies
assignee:YaelDillies
none
16-2360
16 days ago
31-9258
1 month ago
49-66650
49 days
24816 ciskiko
author:ciskiko
feat(GroupTheory): add Regular Wreath Product feat: add regular wreath product and some results; add iterated wreath product; add the isomorphism of iterated wreath product of Z_p to sylow p subgroup of S_{p^n}. Needs some work simplifying final result. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) maintainer-merge new-contributor t-algebra
label:t-algebra$
285/1 Mathlib.lean,Mathlib/Algebra/Group/End.lean,Mathlib/Combinatorics/Additive/AP/Three/Behrend.lean,Mathlib/Data/Nat/Multiplicity.lean,Mathlib/GroupTheory/RegularWreathProduct.lean,Mathlib/Logic/Equiv/Fin/Basic.lean,Mathlib/SetTheory/Cardinal/Finite.lean 7 102 ['ciskiko', 'github-actions', 'tb65536'] tb65536
assignee:tb65536
none
15-33430
15 days ago
15-33431
15 days ago
24-38027
24 days
23161 mans0954
author:mans0954
feature(Data/Finset/RangeDistance): abs_sub_lt_of_mem_finset_range The distance between two elements of `Finset.range N` (i.e. absolute value of the difference as integers) is less than `N`. A lemma I found useful for something I was working on, so sharing here in case it's of wider interest. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data 30/0 Mathlib.lean,Mathlib/Algebra/Order/Group/Unbundled/Abs.lean,Mathlib/Data/Finset/RangeDistance.lean 3 4 ['fbarroero', 'github-actions', 'mans0954'] ericrbg
assignee:ericrbg
none
10-82258
10 days ago
81-2744
2 months ago
81-2735
81 days
22771 alreadydone
author:alreadydone
feat(Homotopy/Lifting): monodromy of a covering map 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 2 ['github-actions', 'mathlib4-dependent-issues-bot'] PatrickMassot
assignee:PatrickMassot
none
6-18915
6 days ago
82-35471
2 months ago
82-37366
82 days
22279 xyzw12345
author:xyzw12345
feat(RingTheory/GradedAlgebra): homogeneous relation In this PR, we defined the concept of a homogeneous relation and proved some properties about homogeneous relations. The main result of this PR is showing that taking `RingQuot` by a homogeneous relation can give a graded structure on the quotient ring. This result can be used to define graded structures on rings obtained using `RingQuot`, e.g. the Symmetric Algebra defined in #21539 can be verified to have such a structure. Co-authored-by: Zhixuan Dai @atstarrysky <22300180006@m.fudan.edu.cn> Yiming Fu @pelicanhere Zhenyan Fu @pumpkin678 Raphael Douglas Giles @Raph-DG Jiedong Jiang @jjdishere - [x] depends on: #22354 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra
label:t-algebra$
455/0 Mathlib.lean,Mathlib/Algebra/Algebra/Equiv.lean,Mathlib/Algebra/DirectSum/Basic.lean,Mathlib/Algebra/DirectSum/Module.lean,Mathlib/Algebra/Module/LinearMap/Defs.lean,Mathlib/Algebra/RingQuot.lean,Mathlib/RingTheory/GradedAlgebra/Basic.lean,Mathlib/RingTheory/GradedAlgebra/HomogeneousRelation.lean 8 7 ['Paul-Lez', 'github-actions', 'grunweg', 'mathlib4-dependent-issues-bot', 'ocfnash', 'xyzw12345'] ocfnash
assignee:ocfnash
none
6-18655
6 days ago
68-51515
2 months ago
69-83302
69 days
22767 robin-carlier
author:robin-carlier
feat(AlgebraicTopology/SimplexCategory): the augmented simplex category This PR defines `AugmentedSimplexCategory` as `WithInitial SimplexCategory`. Using the API in `CategoryTheory.WithTerminal`, we check that functors out of this category (resp. out of its opposite) corresponds to cosimplicial (resp. simplicial) objects, and we link various construction about simplicial objects in terms of this category. --- - [x] depends on : #22658 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory 118/0 Mathlib.lean,Mathlib/AlgebraicTopology/SimplexCategory/Augmented.lean 2 5 ['github-actions', 'joelriou', 'robin-carlier'] joelriou
assignee:joelriou
none
5-81078
5 days ago
20-23280
20 days ago
90-81566
90 days
23935 Thmoas-Guan
author:Thmoas-Guan
feat(RingTheory/IsSMulRegular): categorical constructions for IsSMulRegular The categorical constructions for `IsSMulRegular` for later use related to `Ext` in a separate file. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-category-theory
label:t-algebra$
62/0 Mathlib.lean,Mathlib/Algebra/Homology/ExactSequence.lean,Mathlib/RingTheory/Regular/Category.lean 3 36 ['Thmoas-Guan', 'erdOne', 'github-actions', 'joelriou', 'riccardobrasca'] joelriou
assignee:joelriou
none
4-54006
4 days ago
17-33074
17 days ago
49-76048
49 days
24465 adomani
author:adomani
feat: a linter to enforce formatting This linter enforces that the hypotheses of every declaration are correctly formatted. This already required multiple PRs to make mathlib compliant. Ideally, little by little the linter can be extended to format more of mathlib. --- The default linter option is `false`, but the lakefile enforces it to be `true`. This means that the linter does not run on `MathlibTest`. However, the tests should still be compliant, since the default option was `true` in development and the tests were fixed. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-linter maintainer-merge 876/4 Mathlib.lean,Mathlib/Algebra/Group/Int/Defs.lean,Mathlib/Algebra/Group/Nat/Defs.lean,Mathlib/Algebra/Ring/Int/Defs.lean,Mathlib/Data/FunLike/Basic.lean,Mathlib/Data/SetLike/Basic.lean,Mathlib/Init.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter/CommandStart.lean,Mathlib/Tactic/Simps/NotationClass.lean,MathlibTest/CommandStart.lean,MathlibTest/EuclideanSpace.lean,MathlibTest/Simps.lean,MathlibTest/Traversable.lean,MathlibTest/antidiagonal.lean,MathlibTest/delabLinearIndependent.lean,MathlibTest/matrix.lean,MathlibTest/norm_num.lean,MathlibTest/set_like.lean,MathlibTest/vec_notation.lean 20 89 ['Parcly-Taxel', 'adomani', 'eric-wieser', 'github-actions', 'grunweg', 'leanprover-community-bot-assistant'] grunweg
assignee:grunweg
1
4-30689
4 days ago
27-42382
27 days ago*
40-47103
40 days*
24578 b-mehta
author:b-mehta
feat(Pointwise): cardinality of product set in GroupWithZero This PR: * generalises the assumptions to `card_le_card_image₂_left` and `card_le_card_image₂_right` and golf these: they previously required injectivity everywhere despite using it in only one place. (These lemmas were also used in exactly one place each in mathlib) * adds `card_le_card_mul_left_of_injective` and `card_le_card_mul_right_of_injective` which generalise the typeclass assumptions on the existing `card_le_card_mul_left` and `card_le_card_mul_right` * uses the above to add versions of `card_le_card_mul_left` and `card_le_card_mul_right` in groups with zero. This is useful for applying the pointwise constructions to fields In fact, the first versions of all the above lemmas were written in this generality, but that was seemingly lost during an upstream. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
54/16 Mathlib/Algebra/Group/Pointwise/Finset/Basic.lean,Mathlib/Algebra/GroupWithZero/Pointwise/Finset.lean,Mathlib/Data/Finset/NAry.lean 3 1 ['github-actions'] mariainesdff
assignee:mariainesdff
none
2-20790
2 days ago
32-33368
1 month ago
36-70971
36 days
23502 Timeroot
author:Timeroot
feat(ModelTheory/Semantics): BoundedFormula.realize_foldr_imp Two lemmas for `realize`ing a `BoundedFormula`. --- Pulled out from #19695. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-logic 20/0 Mathlib/ModelTheory/Semantics.lean,Mathlib/ModelTheory/Syntax.lean 2 2 ['Timeroot', 'github-actions'] fpvandoorn
assignee:fpvandoorn
none
1-19362
1 day ago
70-16572
2 months ago
70-16623
70 days
24144 joelriou
author:joelriou
feat(CategoryTheory): the derived adjunction between absolute derived functors An adjunction between functors induces an adjunction between the corresponding left/right derived functors, when these derived functors are *absolute*, i.e. they remain derived functors after the post-composition with any functor. This theorem is the generalized version by Georges Maltsiniotis (*Le théorème de Quillen, d'adjonction des foncteurs dérivés, revisité*, C. R. Math. Acad. Sci. Paris 344 (2007), no. 9) of a theorem by Quillen for adjunctions between model categories. --- - [x] depends on: #24142 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory 159/0 Mathlib.lean,Mathlib/CategoryTheory/Functor/Derived/Adjunction.lean,docs/references.bib 3 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] adamtopaz
assignee:adamtopaz
none
1-14703
1 day ago
22-81104
22 days ago
22-81087
22 days
23849 chrisflav
author:chrisflav
feat(Data/Set): add `Set.encard_iUnion` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data 65/0 Mathlib/Algebra/BigOperators/Finprod.lean,Mathlib/Data/Set/Card/Arithmetic.lean,Mathlib/Data/Set/Finite/Lattice.lean 3 11 ['YaelDillies', 'chrisflav', 'github-actions'] YaelDillies
assignee:YaelDillies
none
0-42428
11 hours ago
31-25784
1 month ago
61-54575
61 days
24520 chrisflav
author:chrisflav
feat(Algebra/Pi): add various `AlgEquiv`s and `RingEquiv`s Add - `RingEquiv.sumArrowEquivProdArrow`: ring version of `Equiv.sumArrowEquivProdArrow`. - `AlgEquiv.sumArrowEquivProdArrow`: algebra version of `Equiv.sumArrowEquivProdArrow`. - `AlgEquiv.piCongrLeft'`: algebra version of `Equiv.piCongrLeft`. - `AlgEquiv.piCongrLeft`: algebra version of `Equiv.piCongrLeft`. - `AlgEquiv.funUnique`: algebra version of `Equiv.funUnique`. - `AlgEquiv.prodCongr`: algebra version of `Equiv.prodCongr`. The four last ones already have ring versions. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
116/1 Mathlib/Algebra/Algebra/Pi.lean,Mathlib/Algebra/Algebra/Prod.lean,Mathlib/Algebra/Ring/Equiv.lean 3 20 ['Ruben-VandeVelde', 'chrisflav', 'eric-wieser', 'github-actions', 'mistarro'] eric-wieser
assignee:eric-wieser
none
0-38754
10 hours ago
15-76048
15 days ago
39-8351
39 days

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

There are currently no PRs with just an infrastructure-related CI failure. Congratulations!

PRs addressing technical debt

Number Author Title Description Labels +/- Modified files (first 100) 📝 💬 All users who commented or reviewed Assignee(s) Updated Last status change total time in review
25161 BoltonBailey
author:BoltonBailey
chore(Algebra/Squarefree/Basic): fix erw This PR addresses an instance of the `erw` linter in `Algebra/Squarefree/Basic` by adding a `squarefree_def` theorem and using this to isolate the implementation. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) tech debt t-algebra awaiting-author
label:t-algebra$
4/1 Mathlib/Algebra/Squarefree/Basic.lean 1 3 ['b-mehta', 'eric-wieser', 'github-actions'] nobody
11-57924
11 days ago
11-57924
11 days ago
4-35623
4 days
25556 Parcly-Taxel
author:Parcly-Taxel
chore: remove >6 month old material in `Deprecated` file-removed tech debt 0/250 Mathlib.lean,Mathlib/Deprecated/Cardinal/Continuum.lean,Mathlib/Deprecated/Cardinal/Finite.lean,Mathlib/Deprecated/Cardinal/PartENat.lean,Mathlib/Deprecated/Order.lean 5 1 ['github-actions'] nobody
2-55793
2 days ago
2-55846
2 days ago
2-55905
2 days
25580 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 134/125 Mathlib/AlgebraicTopology/DoldKan/Decomposition.lean,Mathlib/AlgebraicTopology/DoldKan/Degeneracies.lean,Mathlib/AlgebraicTopology/DoldKan/NCompGamma.lean,Mathlib/AlgebraicTopology/DoldKan/Projections.lean,Mathlib/AlgebraicTopology/SimplexCategory/MorphismProperty.lean,Mathlib/AlgebraicTopology/SimplicialObject/Split.lean,Mathlib/AlgebraicTopology/SimplicialSet/Degenerate.lean,Mathlib/AlgebraicTopology/SimplicialSet/NerveAdjunction.lean,Mathlib/AlgebraicTopology/SimplicialSet/StdSimplex.lean,Mathlib/CategoryTheory/Abelian/GrothendieckCategory/EnoughInjectives.lean,Mathlib/CategoryTheory/Abelian/GrothendieckCategory/Subobject.lean,Mathlib/CategoryTheory/Action/Concrete.lean,Mathlib/CategoryTheory/Action/Monoidal.lean,Mathlib/CategoryTheory/ComposableArrows.lean,Mathlib/CategoryTheory/Extensive.lean,Mathlib/CategoryTheory/Filtered/Basic.lean,Mathlib/CategoryTheory/Galois/Decomposition.lean,Mathlib/CategoryTheory/Galois/EssSurj.lean,Mathlib/CategoryTheory/Limits/Shapes/Equalizers.lean,Mathlib/CategoryTheory/Limits/Shapes/SequentialProduct.lean,Mathlib/CategoryTheory/Limits/Types/Colimits.lean,Mathlib/CategoryTheory/Limits/VanKampen.lean,Mathlib/CategoryTheory/Quotient.lean,Mathlib/CategoryTheory/Sites/Sheaf.lean,Mathlib/CategoryTheory/Subobject/Basic.lean,Mathlib/CategoryTheory/Subobject/FactorThru.lean,Mathlib/CategoryTheory/Subobject/Lattice.lean,Mathlib/CategoryTheory/Triangulated/TStructure/Basic.lean 28 3 ['Parcly-Taxel', 'eric-wieser', 'github-actions'] nobody
1-30932
1 day ago
1-57008
1 day ago
1-56994
1 day
22603 pechersky
author:pechersky
chore(Topology): rename pi family from π to X Only in files that mentioned such a family, via a script: ``` git grep -e "π : . → Type" --name-only | rg Topology | xargs -I{} sed -i -e 's/π/X/g' {} ``` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) tech debt t-topology 238/238 Mathlib/Topology/AlexandrovDiscrete.lean,Mathlib/Topology/Algebra/InfiniteSum/Constructions.lean,Mathlib/Topology/Algebra/Module/Equiv.lean,Mathlib/Topology/Algebra/Order/LiminfLimsup.lean,Mathlib/Topology/Bases.lean,Mathlib/Topology/Bornology/Constructions.lean,Mathlib/Topology/Connected/Basic.lean,Mathlib/Topology/Connected/Clopen.lean,Mathlib/Topology/Connected/LocallyConnected.lean,Mathlib/Topology/Connected/TotallyDisconnected.lean,Mathlib/Topology/Constructions.lean,Mathlib/Topology/ContinuousOn.lean,Mathlib/Topology/EMetricSpace/Diam.lean,Mathlib/Topology/EMetricSpace/Pi.lean,Mathlib/Topology/ExtremallyDisconnected.lean,Mathlib/Topology/Inseparable.lean,Mathlib/Topology/MetricSpace/Basic.lean,Mathlib/Topology/MetricSpace/Infsep.lean,Mathlib/Topology/MetricSpace/ProperSpace.lean,Mathlib/Topology/MetricSpace/Pseudo/Pi.lean,Mathlib/Topology/Metrizable/Basic.lean,Mathlib/Topology/Order/Basic.lean,Mathlib/Topology/Separation/Hausdorff.lean,Mathlib/Topology/UniformSpace/Ascoli.lean 24 1 ['github-actions'] nobody
0-66274
18 hours ago
0-66296
18 hours ago
6-59911
6 days
23676 Parcly-Taxel
author:Parcly-Taxel
chore: deprime `induction` for localizations and quotients All these removed instances of `induction'` generate only one subgoal. In some cases `obtain` can be used. The relevant instances were identified by adding the following to `Mathlib.Tactic.Cases` ```diff diff --git a/Mathlib/Tactic/Cases.lean b/Mathlib/Tactic/Cases.lean index 4a60db6c551..08c06520879 100644 --- a/Mathlib/Tactic/Cases.lean +++ b/Mathlib/Tactic/Cases.lean @@ -122,6 +122,16 @@ elab (name := induction') "induction' " tgts:(Parser.Tactic.elimTarget,+) g.assign result.elimApp let subgoals ← ElimApp.evalNames elimInfo result.alts withArg (generalized := fvarIds) (toClear := targetFVarIds) (toTag := toTag) + let body ← inferType targets[0]! + let names : Array Format := if withArg.1.getArgs.size > 1 then + (withArg.1.getArgs[1]!).getArgs.map Syntax.prettyPrint else Array.empty + let gens : Array Format := if genArg.1.getArgs.size > 1 then + (genArg.1.getArgs[1]!).getArgs.map Syntax.prettyPrint else Array.empty + let inductor : Format := if usingArg.1.getArgs.size > 1 then + Syntax.prettyPrint usingArg.1.getArgs[1]! else "~" + if subgoals.toList.length ≤ 1 then + logInfoAt tgts m!"{body.getAppFn.setPPExplicit true} {inductor} {gens} {names} \ + {subgoals.toList.length}" setGoals <| (subgoals ++ result.others).toList ++ gs /-- The `cases'` tactic is similar to the `cases` tactic in Lean 4 core, but the syntax for giving ``` and then examining [the output](https://github.com/leanprover-community/mathlib4/actions/runs/14270845291/job/40003467676). tech debt 71/77 Mathlib/Algebra/Module/LocalizedModule/Basic.lean,Mathlib/Algebra/Pointwise/Stabilizer.lean,Mathlib/Analysis/SpecialFunctions/Complex/Circle.lean,Mathlib/Analysis/SpecialFunctions/Pow/NNReal.lean,Mathlib/CategoryTheory/Action/Concrete.lean,Mathlib/CategoryTheory/Galois/EssSurj.lean,Mathlib/CategoryTheory/Limits/Types/Colimits.lean,Mathlib/CategoryTheory/Subobject/Basic.lean,Mathlib/CategoryTheory/Subobject/FactorThru.lean,Mathlib/CategoryTheory/Subobject/Lattice.lean,Mathlib/Data/Finset/NoncommProd.lean,Mathlib/Data/Finsupp/BigOperators.lean,Mathlib/Data/Fintype/Quotient.lean,Mathlib/Data/List/Cycle.lean,Mathlib/Data/Nat/ChineseRemainder.lean,Mathlib/Data/Setoid/Partition.lean,Mathlib/GroupTheory/Perm/Sign.lean,Mathlib/RingTheory/OreLocalization/Basic.lean,Mathlib/RingTheory/OreLocalization/Ring.lean 19 11 ['Parcly-Taxel', 'apnelson1', 'eric-wieser', 'github-actions', 'grunweg', 'leanprover-community-bot-assistant', 'urkud'] nobody
0-51824
14 hours ago
2-794
2 days ago
63-65172
63 days
25617 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 88/79 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/Synonym.lean 14 1 ['github-actions'] nobody
0-32126
8 hours ago
0-42925
11 hours ago
0-42910
11 hours
12879 grunweg
author:grunweg
feat: port ge_or_gt linter from mathlib3 Code works and is essentially green: next step is to split up into separate PRs. Feedback welcome on whether: - all the test changes are good, or I should simply allow it in more cases - if calc blocks need to be explicitly exempt --- - [ ] depends on: #12933 - [ ] depends on: #12934 - [ ] depends on: #12931 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) tech debt t-linter merge-conflict blocked-by-other-PR 736/319 Archive/Imo/Imo1960Q1.lean,Archive/Imo/Imo1962Q1.lean,Archive/Imo/Imo1988Q6.lean,Archive/Imo/Imo1994Q1.lean,Archive/Imo/Imo2001Q2.lean,Archive/Imo/Imo2005Q3.lean,Archive/Imo/Imo2006Q3.lean,Archive/Imo/Imo2008Q2.lean,Archive/Imo/Imo2008Q3.lean,Archive/Imo/Imo2008Q4.lean,Archive/Imo/Imo2011Q5.lean,Archive/Imo/Imo2019Q4.lean,Archive/Sensitivity.lean,Archive/Wiedijk100Theorems/AreaOfACircle.lean,Archive/Wiedijk100Theorems/BallotProblem.lean,Archive/Wiedijk100Theorems/BirthdayProblem.lean,Archive/Wiedijk100Theorems/CubingACube.lean,Mathlib.lean,Mathlib/Algebra/DualNumber.lean,Mathlib/Algebra/Order/CauSeq/BigOperators.lean,Mathlib/Algebra/Order/Field/Basic.lean,Mathlib/Algebra/Order/Ring/Defs.lean,Mathlib/Algebra/Polynomial/Basic.lean,Mathlib/Algebra/Polynomial/Degree/Definitions.lean,Mathlib/Algebra/Star/CHSH.lean,Mathlib/Analysis/Analytic/Basic.lean,Mathlib/Analysis/Calculus/UniformLimitsDeriv.lean,Mathlib/Analysis/Complex/Hadamard.lean,Mathlib/Analysis/Complex/UpperHalfPlane/Basic.lean,Mathlib/Analysis/InnerProductSpace/Projection.lean,Mathlib/Analysis/Normed/Group/ControlledClosure.lean,Mathlib/Analysis/NormedSpace/MStructure.lean,Mathlib/Analysis/SpecialFunctions/Log/Base.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Basic.lean,Mathlib/Combinatorics/SimpleGraph/DegreeSum.lean,Mathlib/Combinatorics/SimpleGraph/LapMatrix.lean,Mathlib/Computability/AkraBazzi/AkraBazzi.lean,Mathlib/Computability/AkraBazzi/GrowsPolynomially.lean,Mathlib/Data/Complex/Basic.lean,Mathlib/Data/FP/Basic.lean,Mathlib/Data/Finset/Basic.lean,Mathlib/Data/Finset/Fold.lean,Mathlib/Data/Finsupp/Notation.lean,Mathlib/Data/Int/Lemmas.lean,Mathlib/Data/Nat/Dist.lean,Mathlib/Data/Nat/Lattice.lean,Mathlib/Data/Nat/Parity.lean,Mathlib/Data/Nat/Upto.lean,Mathlib/Data/Ordmap/Ordset.lean,Mathlib/Data/PNat/Basic.lean,Mathlib/Data/UInt.lean,Mathlib/GroupTheory/Coxeter/Length.lean,Mathlib/MeasureTheory/Constructions/Polish.lean,Mathlib/MeasureTheory/Covering/Besicovitch.lean,Mathlib/MeasureTheory/Covering/Vitali.lean,Mathlib/MeasureTheory/Covering/VitaliFamily.lean,Mathlib/MeasureTheory/Integral/Layercake.lean,Mathlib/NumberTheory/LegendreSymbol/JacobiSymbol.lean,Mathlib/NumberTheory/Padics/Hensel.lean,Mathlib/NumberTheory/Padics/PadicNorm.lean,Mathlib/NumberTheory/PellMatiyasevic.lean,Mathlib/NumberTheory/Rayleigh.lean,Mathlib/Order/Filter/AtTopBot.lean,Mathlib/Probability/Process/Stopping.lean,Mathlib/RingTheory/Adjoin/Basic.lean,Mathlib/RingTheory/Polynomial/Basic.lean,Mathlib/SetTheory/Ordinal/Notation.lean,Mathlib/Tactic.lean,Mathlib/Tactic/CancelDenoms/Core.lean,Mathlib/Tactic/Common.lean,Mathlib/Tactic/IntervalCases.lean,Mathlib/Tactic/Linarith/Datatypes.lean,Mathlib/Tactic/Linarith/Lemmas.lean,Mathlib/Tactic/Linarith/Oracle/FourierMotzkin.lean,Mathlib/Tactic/Linter/GeOrGt.lean,Mathlib/Tactic/Linter/Style.lean,Mathlib/Tactic/NormNum/GCD.lean,Mathlib/Tactic/NormNum/Inv.lean,Mathlib/Tactic/Ring/Basic.lean,Mathlib/Topology/Category/Profinite/Nobeling.lean,Mathlib/Topology/ContinuousFunction/Bounded.lean,Mathlib/Topology/MetricSpace/CauSeqFilter.lean,Mathlib/Topology/MetricSpace/Cauchy.lean,Mathlib/Topology/MetricSpace/Closeds.lean,Mathlib/Topology/Sequences.lean,scripts/lint-style.py,test/Explode.lean,test/GCongr/inequalities.lean,test/GeOrGt.lean,test/LibrarySearch/IsCompact.lean,test/LibrarySearch/basic.lean,test/Recall.lean,test/Rify.lean,test/Use.lean,test/cancel_denoms.lean,test/congr.lean,test/delabLinearIndependent.lean,test/delaborators.lean,test/interval_cases.lean,test/linarith.lean 109 3 ['github-actions', 'grunweg', 'leanprover-community-mathlib4-bot'] nobody
313-42770
10 months ago
335-23470
11 months ago
0-15202
4 hours
13791 digama0
author:digama0
refactor: Primrec and Partrec General cleanup of the `Primrec` and `Partrec` files, to better adjust to lean 4 things. The main user-visible change is that `Primrec₂` is no longer a `def` but an `abbrev`, because it was causing inference issues in lean 4. I also removed all the nonterminal `simp`s in `PartrecCode.lean`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) tech debt t-computability merge-conflict 585/778 Mathlib/Computability/Ackermann.lean,Mathlib/Computability/Halting.lean,Mathlib/Computability/Partrec.lean,Mathlib/Computability/PartrecCode.lean,Mathlib/Computability/Primrec.lean 5 2 ['github-actions', 'grunweg'] nobody
294-85555
9 months ago
335-23470
11 months ago
1-84718
1 day
15448 urkud
author:urkud
chore(*): deprecate `Option.elim'` Use `Option.elim` instead. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) tech debt merge-conflict awaiting-author 54/50 Mathlib/Algebra/BigOperators/Option.lean,Mathlib/Algebra/MvPolynomial/Equiv.lean,Mathlib/Algebra/MvPolynomial/Variables.lean,Mathlib/Analysis/BoxIntegral/Partition/Additive.lean,Mathlib/Analysis/BoxIntegral/Partition/Basic.lean,Mathlib/Analysis/BoxIntegral/Partition/Split.lean,Mathlib/Analysis/Calculus/LagrangeMultipliers.lean,Mathlib/CategoryTheory/Category/PartialFun.lean,Mathlib/Computability/TMToPartrec.lean,Mathlib/Data/Option/Defs.lean,Mathlib/LinearAlgebra/Basis.lean,Mathlib/Logic/Embedding/Set.lean,Mathlib/Logic/Equiv/Basic.lean,Mathlib/MeasureTheory/OuterMeasure/Induced.lean,Mathlib/NumberTheory/Dioph.lean,Mathlib/Topology/Compactness/Paracompact.lean,Mathlib/Topology/LocallyFinite.lean 17 12 ['Ruben-VandeVelde', 'YaelDillies', 'github-actions', 'grunweg', 'urkud'] nobody
294-9120
9 months ago
294-84667
9 months ago
7-18420
7 days
16464 Parcly-Taxel
author:Parcly-Taxel
chore: deprecate `Nat.(case_)strong_induction_on` …in favour of the now-renamed `Nat.(case)strongInductionOn` in core. tech debt merge-conflict 54/56 Archive/Imo/Imo1981Q3.lean,Mathlib/Algebra/ContinuedFractions/Computation/Approximations.lean,Mathlib/Algebra/ContinuedFractions/Computation/TerminatesIffRat.lean,Mathlib/Algebra/ContinuedFractions/ConvergentsEquiv.lean,Mathlib/Algebra/Polynomial/Derivative.lean,Mathlib/Algebra/Polynomial/Lifts.lean,Mathlib/Analysis/Analytic/Basic.lean,Mathlib/Analysis/Calculus/ContDiff/Bounds.lean,Mathlib/Analysis/Hofer.lean,Mathlib/Analysis/SpecificLimits/Normed.lean,Mathlib/Combinatorics/Derangements/Finite.lean,Mathlib/Combinatorics/Enumerative/Catalan.lean,Mathlib/Combinatorics/Hall/Finite.lean,Mathlib/Combinatorics/SetFamily/AhlswedeZhang.lean,Mathlib/Computability/Primrec.lean,Mathlib/Data/Fintype/Basic.lean,Mathlib/Data/Fintype/Card.lean,Mathlib/Data/Nat/Choose/Central.lean,Mathlib/Data/Nat/Defs.lean,Mathlib/Data/Nat/Digits.lean,Mathlib/Data/Nat/Log.lean,Mathlib/FieldTheory/Separable.lean,Mathlib/LinearAlgebra/Eigenspace/Triangularizable.lean,Mathlib/LinearAlgebra/Multilinear/Basic.lean,Mathlib/NumberTheory/BernoulliPolynomials.lean,Mathlib/NumberTheory/DiophantineApproximation.lean,Mathlib/NumberTheory/Pell.lean,Mathlib/NumberTheory/Primorial.lean,Mathlib/Order/Fin/Basic.lean,Mathlib/RingTheory/Adjoin/PowerBasis.lean,Mathlib/RingTheory/LittleWedderburn.lean,Mathlib/RingTheory/Polynomial/Basic.lean,Mathlib/RingTheory/Polynomial/Cyclotomic/Basic.lean,Mathlib/RingTheory/Polynomial/Cyclotomic/Eval.lean,Mathlib/RingTheory/Polynomial/Eisenstein/IsIntegral.lean,Mathlib/RingTheory/Polynomial/Nilpotent.lean,Mathlib/RingTheory/PowerSeries/Basic.lean,Mathlib/RingTheory/QuotientNilpotent.lean,Mathlib/RingTheory/WittVector/Defs.lean,Mathlib/RingTheory/WittVector/Frobenius.lean,Mathlib/RingTheory/WittVector/StructurePolynomial.lean,Mathlib/SetTheory/Surreal/Dyadic.lean,Mathlib/Topology/Metrizable/Uniformity.lean 43 13 ['Parcly-Taxel', 'b-mehta', 'github-actions', 'jcommelin'] nobody
262-8623
8 months ago
262-8623
8 months ago
8-1989
8 days
20872 grunweg
author:grunweg
feat: lint against the tactic.skipAssignedInstances option in mathlib This means we can remove the corresponding technical debt entry. We also correct some outdated details in the Linter/Style.lean docstring. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) tech debt t-linter merge-conflict awaiting-author 63/7 Mathlib/Analysis/InnerProductSpace/PiL2.lean,Mathlib/Tactic/Linter/Style.lean,Mathlib/Topology/Separation/Regular.lean,MathlibTest/LintStyle.lean,scripts/technical-debt-metrics.sh 5 17 ['adomani', 'github-actions', 'grunweg'] nobody
130-84729
4 months ago
130-84729
4 months ago
0-9411
2 hours
22682 grunweg
author:grunweg
chore(Topology/Homeomorph): split out various constructions This makes `Homeomorph.lean` slightly more manageable, and also is a mild import reduction. edit: also split out IsHomeomorph, as this allows removing the dependencies on Constructions. Let's see if this gains much --- I don't feel strongly about this PR, but we might as well take it. - [ ] depends on: #22681 - [ ] depends on #22827 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) tech debt t-topology RFC merge-conflict 341/290 Mathlib.lean,Mathlib/Topology/Category/TopCat/ULift.lean,Mathlib/Topology/Homeomorph/Constructions.lean,Mathlib/Topology/Homeomorph/IsHomeomorph.lean,Mathlib/Topology/Homeomorph/Lemmas.lean,Mathlib/Topology/NoetherianSpace.lean 6 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
69-57349
2 months ago
69-57349
2 months ago
14-35834
14 days
23411 PatrickMassot
author:PatrickMassot
chore: remove finiteness from Order.Filter.Lift Co-authored-by: Anatole Dedecker --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) longest-pole t-topology merge-conflict 48/21 Mathlib/Dynamics/TopologicalEntropy/DynamicalEntourage.lean,Mathlib/Order/Filter/Basic.lean,Mathlib/Order/Filter/Finite.lean,Mathlib/Order/Filter/Lift.lean,Mathlib/Order/Filter/SmallSets.lean,Mathlib/Topology/Algebra/ContinuousMonoidHom.lean,Mathlib/Topology/Basic.lean 7 4 ['Vierkantor', 'github-actions', 'kim-em', 'leanprover-community-bot-assistant'] nobody
62-38370
2 months ago
62-57939
2 months ago
10-21608
10 days
23211 Parcly-Taxel
author:Parcly-Taxel
chore: automatically deprime common `induction'` uses Replace `induction'` with `induction` for the following targets: ```python rep_dict = {("Nat", "~", 2): [("zero", 0), ("succ", 2)], ("Nat", "strong_induction_on", 1): [("h", 2)], ("Nat", "case_strong_induction_on", 2): [("hz", 0), ("hi", 2)], ("Nat", "le_induction", 2): [("base", 0), ("succ", 3)], ("List", "~", 2): [("nil", 0), ("cons", 3)], ("List", "reverseRecOn", 2): [("nil", 0), ("append_singleton", 3)], ("Multiset", "induction_on", 2): [("empty", 0), ("cons", 3)], ("Finset", "induction", 2): [("empty", 0), ("@insert", 4)], ("Finset", "induction_on", 2): [("empty", 0), ("@insert", 4)], ("MvPolynomial", "induction_on'", 2): [("monomial", 2), ("add", 4)], ("MvPolynomial", "induction_on", 3): [("C", 1), ("add", 4), ("mul_X", 3)]} ``` The script and the data file used can be found [here](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/The.20plan.20to.20remove.20induction'/near/508218834). tech debt merge-conflict 2189/1565 Archive/Imo/Imo1977Q6.lean,Archive/Imo/Imo2006Q5.lean,Archive/Imo/Imo2013Q1.lean,Archive/Imo/Imo2013Q5.lean,Archive/Imo/Imo2019Q4.lean,Archive/Imo/Imo2024Q1.lean,Archive/MiuLanguage/DecisionSuf.lean,Archive/Sensitivity.lean,Archive/Wiedijk100Theorems/FriendshipGraphs.lean,Archive/Wiedijk100Theorems/Partition.lean,Mathlib/Algebra/Algebra/Subalgebra/Lattice.lean,Mathlib/Algebra/BigOperators/Group/List/Lemmas.lean,Mathlib/Algebra/Group/Conj.lean,Mathlib/Algebra/Group/ForwardDiff.lean,Mathlib/Algebra/Group/Pointwise/Finset/Basic.lean,Mathlib/Algebra/Group/Pointwise/Set/BigOperators.lean,Mathlib/Algebra/Group/Pointwise/Set/Finite.lean,Mathlib/Algebra/Group/Pointwise/Set/ListOfFn.lean,Mathlib/Algebra/Lie/Solvable.lean,Mathlib/Algebra/Module/PID.lean,Mathlib/Algebra/Order/BigOperators/Group/List.lean,Mathlib/Algebra/Order/CauSeq/BigOperators.lean,Mathlib/Algebra/Order/Group/Multiset.lean,Mathlib/Algebra/Polynomial/BigOperators.lean,Mathlib/Algebra/Polynomial/Degree/Lemmas.lean,Mathlib/Algebra/Polynomial/Derivative.lean,Mathlib/Algebra/Polynomial/EraseLead.lean,Mathlib/Algebra/Polynomial/Eval/Defs.lean,Mathlib/Algebra/Polynomial/HasseDeriv.lean,Mathlib/Algebra/Ring/Subring/Basic.lean,Mathlib/Algebra/Tropical/BigOperators.lean,Mathlib/AlgebraicTopology/DoldKan/Decomposition.lean,Mathlib/AlgebraicTopology/DoldKan/Degeneracies.lean,Mathlib/AlgebraicTopology/DoldKan/Projections.lean,Mathlib/Analysis/Analytic/Composition.lean,Mathlib/Analysis/Analytic/Constructions.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/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/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/Log/Base.lean,Mathlib/Analysis/SpecialFunctions/Pow/Deriv.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/EulerSineProd.lean,Mathlib/CategoryTheory/ComposableArrows.lean,Mathlib/CategoryTheory/Extensive.lean,Mathlib/CategoryTheory/Filtered/Basic.lean,Mathlib/CategoryTheory/Limits/VanKampen.lean,Mathlib/CategoryTheory/Triangulated/TStructure/Basic.lean,Mathlib/Computability/Ackermann.lean,Mathlib/Computability/DFA.lean,Mathlib/Computability/EpsilonNFA.lean,Mathlib/Computability/Language.lean,Mathlib/Computability/NFA.lean,Mathlib/Computability/Partrec.lean,Mathlib/Computability/PartrecCode.lean,Mathlib/Computability/PostTuringMachine.lean,Mathlib/Computability/Primrec.lean,Mathlib/Computability/RegularExpressions.lean,Mathlib/Computability/TMConfig.lean,Mathlib/Computability/TMToPartrec.lean,Mathlib/Computability/Tape.lean,Mathlib/Control/LawfulFix.lean,Mathlib/Data/Complex/Exponential.lean,Mathlib/Data/Countable/Basic.lean,Mathlib/Data/DFinsupp/Defs.lean,Mathlib/Data/DFinsupp/WellFounded.lean,Mathlib/Data/Fin/Tuple/Basic.lean,Mathlib/Data/Fin/Tuple/NatAntidiagonal.lean,Mathlib/Data/Finmap.lean,Mathlib/Data/Finset/Fold.lean,Mathlib/Data/Finset/Image.lean,Mathlib/Data/Finset/Lattice/Fold.lean,Mathlib/Data/Finset/Lattice/Lemmas.lean,Mathlib/Data/Finset/Lattice/Pi.lean,Mathlib/Data/Finset/Max.lean,Mathlib/Data/Finset/NAry.lean,Mathlib/Data/Finset/NoncommProd.lean,Mathlib/Data/Finset/Sym.lean,Mathlib/Data/Finsupp/BigOperators.lean,Mathlib/Data/Fintype/Basic.lean,Mathlib/Data/Fintype/Card.lean,Mathlib/Data/Fintype/EquivFin.lean,Mathlib/Data/Fintype/Fin.lean 283 2 ['github-actions', 'leanprover-community-bot-assistant'] nobody
55-47427
1 month ago
55-47429
1 month ago
10-65025
10 days
22754 Parcly-Taxel
author:Parcly-Taxel
chore: clear more `docBlame` nolints --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import tech debt merge-conflict awaiting-author documentation 78/64 Mathlib/Algebra/CharP/MixedCharZero.lean,Mathlib/Algebra/ContinuedFractions/Computation/Basic.lean,Mathlib/Algebra/EuclideanDomain/Defs.lean,Mathlib/Algebra/Module/Injective.lean,Mathlib/Algebra/Notation/Defs.lean,Mathlib/Algebra/Polynomial/Basic.lean,Mathlib/Analysis/BoxIntegral/Partition/Filter.lean,Mathlib/Data/Analysis/Topology.lean,Mathlib/Data/Stream/Defs.lean,Mathlib/Data/Stream/Init.lean,Mathlib/Geometry/RingedSpace/PresheafedSpace.lean,Mathlib/LinearAlgebra/AffineSpace/AffineEquiv.lean,Mathlib/LinearAlgebra/AffineSpace/AffineMap.lean,Mathlib/LinearAlgebra/AffineSpace/Basis.lean,Mathlib/LinearAlgebra/AffineSpace/Independent.lean,Mathlib/LinearAlgebra/Matrix/Transvection.lean,Mathlib/LinearAlgebra/QuadraticForm/Basic.lean,Mathlib/Logic/Equiv/Defs.lean,Mathlib/NumberTheory/ModularForms/SlashActions.lean,Mathlib/NumberTheory/ModularForms/SlashInvariantForms.lean,Mathlib/Order/Atoms.lean,Mathlib/Order/PrimeIdeal.lean,Mathlib/RingTheory/GradedAlgebra/HomogeneousLocalization.lean,Mathlib/RingTheory/PowerBasis.lean,Mathlib/RingTheory/WittVector/Isocrystal.lean,Mathlib/Topology/MetricSpace/GromovHausdorff.lean,Mathlib/Topology/Order/Hom/Esakia.lean,scripts/nolints.json 28 9 ['Parcly-Taxel', 'github-actions', 'jcommelin', 'leanprover-community-bot-assistant'] nobody
52-5824
1 month ago
52-5826
1 month ago
0-3406
56 minutes
24483 Parcly-Taxel
author:Parcly-Taxel
chore: delete >6 month old deprecations (2024-10) See #24271 for the general pattern of regex used in the first (automated) commit. The date range used in this PR is `2024-10-..`. tech debt merge-conflict 2/1182 Mathlib/Algebra/BigOperators/Group/List/Basic.lean,Mathlib/Algebra/CharP/Two.lean,Mathlib/Algebra/Order/Monoid/Unbundled/WithTop.lean,Mathlib/AlgebraicGeometry/Morphisms/ClosedImmersion.lean,Mathlib/AlgebraicGeometry/Morphisms/Preimmersion.lean,Mathlib/AlgebraicGeometry/Restrict.lean,Mathlib/Analysis/Analytic/Basic.lean,Mathlib/Analysis/Calculus/ContDiff/Basic.lean,Mathlib/Analysis/Calculus/ContDiff/Defs.lean,Mathlib/Analysis/Calculus/Deriv/Basic.lean,Mathlib/Analysis/Calculus/Deriv/Comp.lean,Mathlib/Analysis/Calculus/FDeriv/Basic.lean,Mathlib/Analysis/Calculus/FDeriv/Comp.lean,Mathlib/Analysis/Calculus/LineDeriv/Basic.lean,Mathlib/Analysis/Complex/ReImTopology.lean,Mathlib/Analysis/Complex/UpperHalfPlane/Topology.lean,Mathlib/Analysis/LocallyConvex/WeakOperatorTopology.lean,Mathlib/Analysis/LocallyConvex/WithSeminorms.lean,Mathlib/Analysis/Normed/Operator/Banach.lean,Mathlib/Analysis/Normed/Operator/LinearIsometry.lean,Mathlib/Analysis/NormedSpace/OperatorNorm/NormedSpace.lean,Mathlib/CategoryTheory/Limits/Preserves/Limits.lean,Mathlib/CategoryTheory/Sites/Canonical.lean,Mathlib/Data/ENNReal/Inv.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/Data/List/Flatten.lean,Mathlib/Data/List/SplitBy.lean,Mathlib/Data/Nat/Factorization/Basic.lean,Mathlib/Data/Nat/Factorization/Defs.lean,Mathlib/Data/Nat/Factorization/PrimePow.lean,Mathlib/Data/Set/Subset.lean,Mathlib/FieldTheory/IntermediateField/Adjoin/Algebra.lean,Mathlib/Geometry/Manifold/ContMDiff/Defs.lean,Mathlib/Geometry/Manifold/LocalInvariantProperties.lean,Mathlib/Geometry/Manifold/MFDeriv/Basic.lean,Mathlib/GroupTheory/CosetCover.lean,Mathlib/GroupTheory/GroupAction/Blocks.lean,Mathlib/LinearAlgebra/Eigenspace/Basic.lean,Mathlib/MeasureTheory/Constructions/BorelSpace/Basic.lean,Mathlib/MeasureTheory/Function/StronglyMeasurable/AEStronglyMeasurable.lean,Mathlib/MeasureTheory/Measure/DiracProba.lean,Mathlib/MeasureTheory/Measure/FiniteMeasure.lean,Mathlib/MeasureTheory/Measure/ProbabilityMeasure.lean,Mathlib/NumberTheory/NumberField/Embeddings.lean,Mathlib/Order/InitialSeg.lean,Mathlib/Order/WellFounded.lean,Mathlib/Probability/Density.lean,Mathlib/RingTheory/Finiteness/Cardinality.lean,Mathlib/RingTheory/Finiteness/Ideal.lean,Mathlib/RingTheory/Jacobson/Ring.lean,Mathlib/RingTheory/Localization/Cardinality.lean,Mathlib/RingTheory/PowerSeries/Basic.lean,Mathlib/RingTheory/Spectrum/Prime/TensorProduct.lean,Mathlib/RingTheory/Spectrum/Prime/Topology.lean,Mathlib/SetTheory/Game/Nim.lean,Mathlib/SetTheory/PGame/Algebra.lean,Mathlib/Tactic/FunProp/ContDiff.lean,Mathlib/Topology/AlexandrovDiscrete.lean,Mathlib/Topology/Algebra/ConstMulAction.lean,Mathlib/Topology/Algebra/Constructions.lean,Mathlib/Topology/Algebra/Constructions/DomMulAct.lean,Mathlib/Topology/Algebra/Group/Basic.lean,Mathlib/Topology/Algebra/Group/CompactOpen.lean,Mathlib/Topology/Algebra/Group/Quotient.lean,Mathlib/Topology/Algebra/GroupWithZero.lean,Mathlib/Topology/Algebra/InfiniteSum/Basic.lean,Mathlib/Topology/Algebra/Module/Alternating/Topology.lean,Mathlib/Topology/Algebra/Module/Equiv.lean,Mathlib/Topology/Algebra/Module/Multilinear/Topology.lean,Mathlib/Topology/Algebra/Module/StrongTopology.lean,Mathlib/Topology/Algebra/Module/WeakBilin.lean,Mathlib/Topology/Algebra/Monoid.lean,Mathlib/Topology/Algebra/MulAction.lean,Mathlib/Topology/Algebra/Ring/Ideal.lean,Mathlib/Topology/Algebra/SeparationQuotient/Section.lean,Mathlib/Topology/Algebra/StarSubalgebra.lean,Mathlib/Topology/Bases.lean,Mathlib/Topology/Category/Profinite/Nobeling/Induction.lean,Mathlib/Topology/Category/TopCat/EffectiveEpi.lean,Mathlib/Topology/Category/TopCat/Limits/Products.lean,Mathlib/Topology/Category/TopCat/Limits/Pullbacks.lean,Mathlib/Topology/Clopen.lean,Mathlib/Topology/CompactOpen.lean,Mathlib/Topology/Compactness/Compact.lean,Mathlib/Topology/Compactness/Lindelof.lean,Mathlib/Topology/Compactness/LocallyCompact.lean,Mathlib/Topology/Compactness/SigmaCompact.lean,Mathlib/Topology/Connected/Basic.lean,Mathlib/Topology/Connected/Clopen.lean,Mathlib/Topology/Connected/PathConnected.lean,Mathlib/Topology/Connected/TotallyDisconnected.lean,Mathlib/Topology/Constructions.lean,Mathlib/Topology/Constructions/SumProd.lean,Mathlib/Topology/ContinuousMap/Bounded/Basic.lean,Mathlib/Topology/ContinuousMap/ContinuousMapZero.lean,Mathlib/Topology/ContinuousMap/Sigma.lean,Mathlib/Topology/ContinuousMap/T0Sierpinski.lean,Mathlib/Topology/ContinuousOn.lean,Mathlib/Topology/Covering.lean,Mathlib/Topology/Defs/Induced.lean 139 3 ['github-actions', 'leanprover-community-bot-assistant'] nobody
35-41124
1 month ago
35-41126
1 month ago
4-54091
4 days
24100 eric-wieser
author:eric-wieser
feat: restore some explicit binders from Lean 3 Part of #24099 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) tech debt merge-conflict awaiting-author 39/42 Mathlib/Data/FinEnum.lean,Mathlib/FieldTheory/Galois/Profinite.lean,Mathlib/Topology/Bases.lean,Mathlib/Topology/Compactness/CompactlyGeneratedSpace.lean,Mathlib/Topology/MetricSpace/IsometricSMul.lean,Mathlib/Topology/Metrizable/CompletelyMetrizable.lean,Mathlib/Topology/Metrizable/Uniformity.lean,Mathlib/Topology/Order.lean,Mathlib/Topology/Order/LowerUpperTopology.lean,Mathlib/Topology/UniformSpace/UniformEmbedding.lean 10 3 ['github-actions', 'grunweg', 'leanprover-community-bot-assistant'] nobody
15-21523
15 days ago
15-21525
15 days ago
34-33204
34 days
24409 urkud
author:urkud
chore(*): fix `nmem` vs `not_mem` names --- There are some missing/buggy deprecations, I'm going to fix them later today or tomorrow. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-zulip tech debt merge-conflict delegated awaiting-author 317/176 Mathlib/Algebra/BigOperators/Finprod.lean,Mathlib/Algebra/BigOperators/Group/Finset/Lemmas.lean,Mathlib/Algebra/Group/Indicator.lean,Mathlib/Algebra/Group/Support.lean,Mathlib/Algebra/GroupWithZero/NonZeroDivisors.lean,Mathlib/Algebra/Order/Group/Indicator.lean,Mathlib/Algebra/Polynomial/AlgebraMap.lean,Mathlib/Algebra/Polynomial/Degree/Operations.lean,Mathlib/Analysis/Calculus/BumpFunction/Basic.lean,Mathlib/Analysis/Calculus/DSlope.lean,Mathlib/Analysis/Calculus/Deriv/Basic.lean,Mathlib/Analysis/Calculus/Deriv/Support.lean,Mathlib/Analysis/Calculus/FDeriv/Basic.lean,Mathlib/Analysis/Calculus/Rademacher.lean,Mathlib/Analysis/Complex/RemovableSingularity.lean,Mathlib/Analysis/Convex/Cone/InnerDual.lean,Mathlib/Analysis/Convex/Cone/Proper.lean,Mathlib/Analysis/Convolution.lean,Mathlib/Analysis/Distribution/AEEqOfIntegralContDiff.lean,Mathlib/Data/LocallyFinsupp.lean,Mathlib/Data/Set/Basic.lean,Mathlib/Data/Set/Insert.lean,Mathlib/Dynamics/Ergodic/Conservative.lean,Mathlib/Dynamics/Ergodic/Ergodic.lean,Mathlib/Dynamics/Ergodic/Function.lean,Mathlib/Dynamics/PeriodicPts/Defs.lean,Mathlib/Geometry/Manifold/ContMDiff/Basic.lean,Mathlib/Geometry/Manifold/PartitionOfUnity.lean,Mathlib/GroupTheory/CosetCover.lean,Mathlib/LinearAlgebra/Dual/Lemmas.lean,Mathlib/LinearAlgebra/FreeModule/PID.lean,Mathlib/LinearAlgebra/PID.lean,Mathlib/LinearAlgebra/RootSystem/Base.lean,Mathlib/LinearAlgebra/RootSystem/Finite/Lemmas.lean,Mathlib/MeasureTheory/Function/ContinuousMapDense.lean,Mathlib/MeasureTheory/Function/ConvergenceInMeasure.lean,Mathlib/MeasureTheory/Function/L2Space.lean,Mathlib/MeasureTheory/Function/LocallyIntegrable.lean,Mathlib/MeasureTheory/Function/LpSpace/Indicator.lean,Mathlib/MeasureTheory/Integral/Average.lean,Mathlib/MeasureTheory/Integral/Bochner/Set.lean,Mathlib/MeasureTheory/Integral/Layercake.lean,Mathlib/MeasureTheory/Integral/Lebesgue/Add.lean,Mathlib/MeasureTheory/Integral/Lebesgue/Basic.lean,Mathlib/MeasureTheory/Integral/RieszMarkovKakutani/Basic.lean,Mathlib/MeasureTheory/Integral/RieszMarkovKakutani/Real.lean,Mathlib/MeasureTheory/Measure/AbsolutelyContinuous.lean,Mathlib/MeasureTheory/Measure/AddContent.lean,Mathlib/MeasureTheory/Measure/DiracProba.lean,Mathlib/MeasureTheory/Measure/Haar/Unique.lean,Mathlib/MeasureTheory/Measure/Restrict.lean,Mathlib/MeasureTheory/Measure/WithDensity.lean,Mathlib/MeasureTheory/OuterMeasure/AE.lean,Mathlib/MeasureTheory/SetSemiring.lean,Mathlib/Order/Filter/AtTopBot/CountablyGenerated.lean,Mathlib/Order/Filter/Cocardinal.lean,Mathlib/Order/Filter/Cofinite.lean,Mathlib/Order/Filter/Tendsto.lean,Mathlib/Order/Filter/Ultrafilter/Basic.lean,Mathlib/Probability/Distributions/Uniform.lean,Mathlib/Probability/Kernel/Basic.lean,Mathlib/Probability/Kernel/Composition/MeasureCompProd.lean,Mathlib/RingTheory/AdicCompletion/LocalRing.lean,Mathlib/RingTheory/Ideal/Maximal.lean,Mathlib/RingTheory/LaurentSeries.lean,Mathlib/RingTheory/MvPolynomial/Symmetric/NewtonIdentities.lean,Mathlib/RingTheory/MvPowerSeries/NoZeroDivisors.lean,Mathlib/RingTheory/Spectrum/Maximal/Localization.lean,Mathlib/RingTheory/Spectrum/Prime/RingHom.lean,Mathlib/RingTheory/Spectrum/Prime/Topology.lean,Mathlib/Topology/Algebra/InfiniteSum/Group.lean,Mathlib/Topology/Algebra/Module/Cardinality.lean,Mathlib/Topology/Algebra/Support.lean,Mathlib/Topology/Bases.lean,Mathlib/Topology/ContinuousMap/BoundedCompactlySupported.lean,Mathlib/Topology/Order/Basic.lean,Mathlib/Topology/UrysohnsLemma.lean 77 4 ['b-mehta', 'github-actions', 'jcommelin', 'leanprover-community-bot-assistant', 'mathlib-bors'] nobody
7-49043
7 days ago
7-49043
7 days ago
0-55045
15 hours
23394 BoltonBailey
author:BoltonBailey
chore(Data/Int/WithZero): fix erw --- Removing an `erw`. This is my first time doing this, so please tell me if I am doing something wrong here (e.g. should the new lemma be `simp`?). [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) tech debt merge-conflict 5/4 Mathlib/Algebra/Group/WithOne/Defs.lean,Mathlib/Algebra/GroupWithZero/WithZero.lean,Mathlib/Data/Int/WithZero.lean 3 19 ['BoltonBailey', 'Ruben-VandeVelde', 'eric-wieser', 'fpvandoorn', 'github-actions', 'grunweg', 'leanprover-community-bot-assistant'] nobody
0-50895
14 hours ago
0-50897
14 hours ago
52-38111
52 days

PRs blocked on a zulip discussion

Number Author Title Description Labels +/- Modified files (first 100) 📝 💬 All users who commented or reviewed Assignee(s) Updated Last status change total time in review
23866 kim-em
author:kim-em
chore: remove `[AtLeastTwo n]` hypothesis from the `NatCast` to `OfNat` instance This PR observes that we can change ``` instance (priority := 100) instOfNatAtLeastTwo {n : ℕ} [NatCast R] [Nat.AtLeastTwo n] : OfNat R n ``` to ``` instance (priority := 100) instOfNatAtLeastTwo {n : ℕ} [NatCast R] : OfNat R n ``` with minimal fall-out. A follow-up PR #23867 then observes that we can remove nearly all the `[Nat.AtLeastTwo n]` hypotheses in Mathlib. This is slightly dangerous -- it does make it more likely that we'll generate non-defeq instances, but it appears to happen very rarely. However, it will make life slightly easier for something Leo and I are trying to do with `grind` and Grobner bases (we'd like to be able to assume types we consume have `[∀ n, OfNat α n]`, which is possible with this change, but not without...). Zulip thread: [#PR reviews > #23866 and #23867, removing most `[Nat.AtLeastTwo n]` @ 💬](https://leanprover.zulipchat.com/#narrow/channel/144837-PR-reviews/topic/.2323866.20and.20.2323867.2C.20removing.20most.20.60.5BNat.2EAtLeastTwo.20n.5D.60/near/511157297) awaiting-zulip 21/26 Mathlib/AlgebraicTopology/FundamentalGroupoid/Basic.lean,Mathlib/Data/Nat/Cast/Defs.lean,Mathlib/Data/Nat/Cast/Order/Basic.lean 3 3 ['eric-wieser', 'github-actions', 'urkud'] nobody
61-4028
2 months ago
61-4117
2 months ago
0-23929
6 hours
15649 TpmKranz
author:TpmKranz
feat(Computability): introduce Generalised NFA as bridge to Regular Expression Lays the groundwork for a proof of equivalence of NFA and RE, w.r.t. described language. Actual connection to NFA comes later, after the groundwork for the opposite direction has been laid. Second chunk of #12648 --- - [x] depends on: #15647 [Data.FinEnum.Option unchanged since then] [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-zulip t-computability new-contributor awaiting-author 298/0 Mathlib.lean,Mathlib/Computability/GNFA.lean,Mathlib/Computability/Language.lean,Mathlib/Computability/RegularExpressions.lean,docs/references.bib 5 6 ['github-actions', 'mathlib4-dependent-issues-bot', 'meithecatte', 'trivial1711'] nobody
34-77905
1 month ago
34-77914
1 month ago
23-54870
23 days
20648 anthonyde
author:anthonyde
feat: formalize regular expression -> εNFA The file `Computability/RegularExpressionsToEpsilonNFA.lean` contains a formal definition of Thompson's method for constructing an `εNFA` from a `RegularExpression` and a proof of its correctness. --- - [x] depends on: #20644 - [x] depends on: #20645 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-zulip t-computability new-contributor 490/0 Mathlib.lean,Mathlib/Computability/RegularExpressionsToEpsilonNFA.lean,docs/references.bib 3 5 ['github-actions', 'mathlib4-dependent-issues-bot', 'meithecatte', 'qawbecrdtey'] nobody
34-77216
1 month ago
34-77851
1 month ago
75-77754
75 days
23048 scholzhannah
author:scholzhannah
feat: PartialEquiv on closed sets restricts to closed map This PR shows that a PartialEquiv that is continuous on both source and target restricts to a homeomorphism. It then uses that to show that a PartialEquiv with closed source and target and which is continuous on both the source and target restricts to a closed map. --- See [this Zulip discussion](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Generalizing.20.60PartialHomeomorph.60.3F) that will probably mean that I close this PR. I need the latter statement to prove that one can transport a CW complex along a PartialEquiv. I had trouble finding a good spot for these statements; I hope this solution works. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-zulip t-topology 53/0 Mathlib.lean,Mathlib/Topology/PartialEquiv.lean 2 3 ['ADedecker', 'github-actions', 'scholzhannah'] ADedecker
assignee:ADedecker
27-15400
27 days ago
31-22176
1 month ago
51-86236
51 days
17458 urkud
author:urkud
refactor(Algebra/Group): make `IsUnit` a typeclass Also change some lemmas to assume `[IsUnit _]` instead of `[Invertible _]`. Motivated by potential non-defeq diamonds in #14986, see also [Zulip](https://leanprover.zulipchat.com/#narrow/stream/116395-maths/topic/Invertible.20and.20data) I no longer plan to merge this PR, but I'm going to cherry-pick some changes to a new PR before closing this one. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-zulip t-algebra
label:t-algebra$
82/72 Mathlib/Algebra/CharP/Invertible.lean,Mathlib/Algebra/Group/Invertible/Basic.lean,Mathlib/Algebra/Group/Units/Defs.lean,Mathlib/Algebra/GroupWithZero/Invertible.lean,Mathlib/Algebra/GroupWithZero/Units/Basic.lean,Mathlib/Algebra/Polynomial/Degree/Units.lean,Mathlib/Algebra/Polynomial/Splits.lean,Mathlib/Analysis/Convex/Segment.lean,Mathlib/Analysis/Normed/Affine/Isometry.lean,Mathlib/Analysis/Normed/Ring/Units.lean,Mathlib/CategoryTheory/Linear/Basic.lean,Mathlib/FieldTheory/Finite/Basic.lean,Mathlib/FieldTheory/Separable.lean,Mathlib/FieldTheory/SeparableDegree.lean,Mathlib/GroupTheory/Submonoid/Inverses.lean,Mathlib/LinearAlgebra/AffineSpace/AffineEquiv.lean,Mathlib/LinearAlgebra/AffineSpace/Combination.lean,Mathlib/LinearAlgebra/CliffordAlgebra/Contraction.lean,Mathlib/LinearAlgebra/CliffordAlgebra/Inversion.lean,Mathlib/LinearAlgebra/CliffordAlgebra/SpinGroup.lean,Mathlib/LinearAlgebra/Eigenspace/Minpoly.lean,Mathlib/NumberTheory/MulChar/Basic.lean,Mathlib/RingTheory/Localization/NumDen.lean,Mathlib/RingTheory/Polynomial/Content.lean,Mathlib/RingTheory/Polynomial/GaussLemma.lean,Mathlib/RingTheory/Valuation/Basic.lean 26 11 ['MichaelStollBayreuth', 'acmepjz', 'eric-wieser', 'github-actions', 'leanprover-bot', 'urkud'] nobody
21-63866
21 days ago
21-84293
21 days ago
0-66650
18 hours
20238 maemre
author:maemre
feat(Computability/DFA): Closure of regular languages under some set operations This shows that regular languages are closed under complement and intersection by constructing DFAs for them. --- Closure under all other operations will be proved when someone adds the proof for DFA<->regular expression equivalence, so they are not part of this PR. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-zulip t-computability new-contributor awaiting-author 159/0 Mathlib/Computability/DFA.lean,Mathlib/Computability/Language.lean 2 59 ['EtienneC30', 'YaelDillies', 'github-actions', 'maemre', 'meithecatte', 'urkud'] EtienneC30
assignee:EtienneC30
5-43676
5 days ago
34-77815
1 month ago
48-67492
48 days
25218 kckennylau
author:kckennylau
feat(AlgebraicGeometry): Tate normal form of elliptic curves --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-zulip new-contributor t-algebraic-geometry 291/26 Mathlib.lean,Mathlib/AlgebraicGeometry/EllipticCurve/IsomOfJ.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Modular/TateNormalForm.lean,Mathlib/AlgebraicGeometry/EllipticCurve/NormalForms.lean,Mathlib/AlgebraicGeometry/EllipticCurve/VariableChange.lean 5 29 ['MichaelStollBayreuth', 'Multramate', 'acmepjz', 'github-actions', 'grunweg', 'kckennylau'] nobody
3-79757
3 days ago
7-32169
7 days ago
6-51040
6 days
23658 grunweg
author:grunweg
feat: require that real or complex models with corners have convex interior Follow-up to #18403. --- - [x] depends on: #23657 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-zulip t-differential-geometry WIP 116/18 Mathlib/Geometry/Manifold/Instances/Real.lean,Mathlib/Geometry/Manifold/IsManifold/Basic.lean 2 5 ['github-actions', 'grunweg', 'mathlib4-dependent-issues-bot', 'sgouezel'] nobody
2-31025
2 days ago
6-14472
6 days ago
0-9
9 seconds
23929 meithecatte
author:meithecatte
feat(Computability/NFA): improve bound on pumping lemma --- - [x] depends on: #25321 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-zulip t-computability new-contributor 101/10 Mathlib/Computability/EpsilonNFA.lean,Mathlib/Computability/NFA.lean 2 41 ['YaelDillies', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'meithecatte'] nobody
2-1067
2 days ago
2-1068
2 days ago
34-10595
34 days
11800 JADekker
author:JADekker
feat : Define KappaLindelöf spaces Define KappaLindelöf spaces by following the first one-third of the API for Lindelöf spaces. The remainder will be added in a future PR. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-zulip t-topology merge-conflict please-adopt 301/2 Mathlib.lean,Mathlib/Topology/Compactness/KappaLindelof.lean,Mathlib/Topology/Compactness/Lindelof.lean 3 38 ['ADedecker', 'JADekker', 'PatrickMassot', 'StevenClontz', 'adomani', 'github-actions', 'grunweg', 'kim-em', 'urkud'] nobody
266-54938
8 months ago
266-76913
8 months ago
119-10687
119 days
17518 grunweg
author:grunweg
feat: lint on declarations mentioning `Invertible` or `Unique` Using the same infrastructure as for #10235. Depends on that PR to land first, and also (for the first lint) a zulip discussion if that change is desired/about the best way to enact it. --- - [ ] depends on: #10235 awaiting-zulip t-linter merge-conflict blocked-by-other-PR 149/7 Mathlib.lean,Mathlib/Algebra/MvPolynomial/PDeriv.lean,Mathlib/Computability/Halting.lean,Mathlib/Computability/TuringMachine.lean,Mathlib/Data/Fintype/Card.lean,Mathlib/GroupTheory/Perm/DomMulAct.lean,Mathlib/Logic/Basic.lean,Mathlib/Logic/Encodable/Basic.lean,Mathlib/NumberTheory/JacobiSum/Basic.lean,Mathlib/Order/Heyting/Regular.lean,Mathlib/RingTheory/MvPolynomial/Symmetric/FundamentalTheorem.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter/UnusedAssumptionInType.lean 13 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mergify'] nobody
219-8657
7 months ago
244-83579
8 months ago*
0-0
0 seconds*
17623 FR-vdash-bot
author:FR-vdash-bot
feat(Algebra/Order/GroupWithZero/Unbundled): add some lemmas Some lemmas in `Algebra.Order.GroupWithZero.Unbundled` have incorrect or unsatisfactory names, or assumptions that can be omitted using `ZeroLEOneClass`. The lemmas added in this PR are versions of existing lemmas that use the correct or better name or `ZeroLEOneClass` to omit an assumption. The original lemmas will be deprecated in #17593. | New name | Old name | |-------------------------|-------------------------| | `mul_le_one_left₀` | `Left.mul_le_one_of_le_of_le` | | `mul_lt_one_of_le_of_lt_left₀` (`0 ≤ ·` version) / `mul_lt_one_of_le_of_lt_of_pos_left` | `Left.mul_lt_of_le_of_lt_one_of_pos` | | `mul_lt_one_of_lt_of_le_left₀` | `Left.mul_lt_of_lt_of_le_one_of_nonneg` | | `mul_le_one_right₀` | `Right.mul_le_one_of_le_of_le` | | `mul_lt_one_of_lt_of_le_right₀` (`0 ≤ ·` version) / `mul_lt_one_of_lt_of_le_of_pos_right` | `Right.mul_lt_one_of_lt_of_le_of_pos` | | `mul_lt_one_of_le_of_lt_right₀` | `Right.mul_lt_one_of_le_of_lt_of_nonneg` | The following lemmas use `ZeroLEOneClass`. | New name | Old name | |-------------------------|-------------------------| | `(Left.)one_le_mul₀` | `Left.one_le_mul_of_le_of_le` | | `Left.one_lt_mul_of_le_of_lt₀` | `Left.one_lt_mul_of_le_of_lt_of_pos` | | `Left.one_lt_mul_of_lt_of_le₀` | `Left.lt_mul_of_lt_of_one_le_of_nonneg` / `one_lt_mul_of_lt_of_le` (still there) | | `(Left.)one_lt_mul₀` | | | `Right.one_le_mul₀` | `Right.one_le_mul_of_le_of_le` | | `Right.one_lt_mul_of_lt_of_le₀` | `Right.one_lt_mul_of_lt_of_le_of_pos` | | `Right.one_lt_mul_of_le_of_lt₀` | `Right.one_lt_mul_of_le_of_lt_of_nonneg` / `one_lt_mul_of_le_of_lt` (still there) / `one_lt_mul` (still there) | | `Right.one_lt_mul₀` | `Right.one_lt_mul_of_lt_of_lt` | --- Split from #17593. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-zulip t-order t-algebra merge-conflict
label:t-algebra$
146/44 Mathlib/Algebra/Order/GroupWithZero/Canonical.lean,Mathlib/Algebra/Order/GroupWithZero/Unbundled.lean 2 11 ['FR-vdash-bot', 'YaelDillies', 'github-actions', 'j-loreaux'] nobody
201-28188
6 months ago
201-28188
6 months ago
33-64877
33 days
8370 eric-wieser
author:eric-wieser
refactor(Analysis/NormedSpace/Exponential): remove the `𝕂` argument from `exp` This argument is still needed for almost all the lemmas, which means it can longer be found by unification. We keep around `expSeries 𝕂 A`, as it's needed for talking about the radius of convergence over different base fields. This is a prerequisite for #8372, as we can't merge the functions until they have the same interface.\ Zulip thread: [#mathlib4 > Real.exp @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Real.2Eexp/near/401602245) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) This is started from the mathport output on https://github.com/leanprover-community/mathlib/pull/19244 awaiting-zulip t-analysis merge-conflict 432/387 Mathlib/Analysis/CStarAlgebra/Exponential.lean,Mathlib/Analysis/CStarAlgebra/Spectrum.lean,Mathlib/Analysis/Normed/Algebra/Exponential.lean,Mathlib/Analysis/Normed/Algebra/MatrixExponential.lean,Mathlib/Analysis/Normed/Algebra/QuaternionExponential.lean,Mathlib/Analysis/Normed/Algebra/Spectrum.lean,Mathlib/Analysis/Normed/Algebra/TrivSqZeroExt.lean,Mathlib/Analysis/NormedSpace/DualNumber.lean,Mathlib/Analysis/SpecialFunctions/ContinuousFunctionalCalculus/ExpLog.lean,Mathlib/Analysis/SpecialFunctions/Exponential.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Series.lean 11 29 ['YaelDillies', 'eric-wieser', 'girving', 'github-actions', 'j-loreaux', 'kbuzzard', 'leanprover-community-bot-assistant', 'urkud'] nobody
45-69965
1 month ago
57-12195
1 month ago
29-60989
29 days
15654 TpmKranz
author:TpmKranz
feat(Computability): language-preserving maps between NFA and RE Map REs to NFAs via Thompson's construction and NFAs to REs using GNFAs Last chunk of #12648 --- - [ ] depends on: #15651 - [ ] depends on: #15649 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-zulip t-computability new-contributor merge-conflict blocked-by-other-PR 985/2 Mathlib.lean,Mathlib/Computability/GNFA.lean,Mathlib/Computability/Language.lean,Mathlib/Computability/NFA.lean,Mathlib/Computability/RegularExpressions.lean,Mathlib/Data/FinEnum/Option.lean,docs/references.bib 7 3 ['github-actions', 'leanprover-community-mathlib4-bot', 'meithecatte'] nobody
34-77865
1 month ago
34-77870
1 month ago
0-179
2 minutes
15651 TpmKranz
author:TpmKranz
feat(Computability/NFA): operations for Thompson's construction Lays the groundwork for a proof of equivalence of RE and NFA, w.r.t. described language. Actual connection to REs comes later, after the groundwork for the opposite direction has been laid. Third chunk of #12648 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-zulip t-computability new-contributor merge-conflict awaiting-author 307/5 Mathlib/Computability/NFA.lean 1 15 ['TpmKranz', 'YaelDillies', 'dupuisf', 'github-actions', 'leanprover-community-bot-assistant', 'meithecatte'] nobody
21-14071
21 days ago
21-14072
21 days ago
45-84611
45 days
22361 rudynicolop
author:rudynicolop
feat(Computability/NFA): nfa closure properties Add the closure properties union, intersection and reversal for NFA. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-zulip t-computability new-contributor merge-conflict awaiting-author 218/2 Mathlib/Computability/Language.lean,Mathlib/Computability/NFA.lean 2 90 ['EtienneC30', 'b-mehta', 'github-actions', 'leanprover-community-bot-assistant', 'meithecatte', 'rudynicolop'] EtienneC30
assignee:EtienneC30
21-13145
21 days ago
21-13147
21 days ago
39-67601
39 days
24409 urkud
author:urkud
chore(*): fix `nmem` vs `not_mem` names --- There are some missing/buggy deprecations, I'm going to fix them later today or tomorrow. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-zulip tech debt merge-conflict delegated awaiting-author 317/176 Mathlib/Algebra/BigOperators/Finprod.lean,Mathlib/Algebra/BigOperators/Group/Finset/Lemmas.lean,Mathlib/Algebra/Group/Indicator.lean,Mathlib/Algebra/Group/Support.lean,Mathlib/Algebra/GroupWithZero/NonZeroDivisors.lean,Mathlib/Algebra/Order/Group/Indicator.lean,Mathlib/Algebra/Polynomial/AlgebraMap.lean,Mathlib/Algebra/Polynomial/Degree/Operations.lean,Mathlib/Analysis/Calculus/BumpFunction/Basic.lean,Mathlib/Analysis/Calculus/DSlope.lean,Mathlib/Analysis/Calculus/Deriv/Basic.lean,Mathlib/Analysis/Calculus/Deriv/Support.lean,Mathlib/Analysis/Calculus/FDeriv/Basic.lean,Mathlib/Analysis/Calculus/Rademacher.lean,Mathlib/Analysis/Complex/RemovableSingularity.lean,Mathlib/Analysis/Convex/Cone/InnerDual.lean,Mathlib/Analysis/Convex/Cone/Proper.lean,Mathlib/Analysis/Convolution.lean,Mathlib/Analysis/Distribution/AEEqOfIntegralContDiff.lean,Mathlib/Data/LocallyFinsupp.lean,Mathlib/Data/Set/Basic.lean,Mathlib/Data/Set/Insert.lean,Mathlib/Dynamics/Ergodic/Conservative.lean,Mathlib/Dynamics/Ergodic/Ergodic.lean,Mathlib/Dynamics/Ergodic/Function.lean,Mathlib/Dynamics/PeriodicPts/Defs.lean,Mathlib/Geometry/Manifold/ContMDiff/Basic.lean,Mathlib/Geometry/Manifold/PartitionOfUnity.lean,Mathlib/GroupTheory/CosetCover.lean,Mathlib/LinearAlgebra/Dual/Lemmas.lean,Mathlib/LinearAlgebra/FreeModule/PID.lean,Mathlib/LinearAlgebra/PID.lean,Mathlib/LinearAlgebra/RootSystem/Base.lean,Mathlib/LinearAlgebra/RootSystem/Finite/Lemmas.lean,Mathlib/MeasureTheory/Function/ContinuousMapDense.lean,Mathlib/MeasureTheory/Function/ConvergenceInMeasure.lean,Mathlib/MeasureTheory/Function/L2Space.lean,Mathlib/MeasureTheory/Function/LocallyIntegrable.lean,Mathlib/MeasureTheory/Function/LpSpace/Indicator.lean,Mathlib/MeasureTheory/Integral/Average.lean,Mathlib/MeasureTheory/Integral/Bochner/Set.lean,Mathlib/MeasureTheory/Integral/Layercake.lean,Mathlib/MeasureTheory/Integral/Lebesgue/Add.lean,Mathlib/MeasureTheory/Integral/Lebesgue/Basic.lean,Mathlib/MeasureTheory/Integral/RieszMarkovKakutani/Basic.lean,Mathlib/MeasureTheory/Integral/RieszMarkovKakutani/Real.lean,Mathlib/MeasureTheory/Measure/AbsolutelyContinuous.lean,Mathlib/MeasureTheory/Measure/AddContent.lean,Mathlib/MeasureTheory/Measure/DiracProba.lean,Mathlib/MeasureTheory/Measure/Haar/Unique.lean,Mathlib/MeasureTheory/Measure/Restrict.lean,Mathlib/MeasureTheory/Measure/WithDensity.lean,Mathlib/MeasureTheory/OuterMeasure/AE.lean,Mathlib/MeasureTheory/SetSemiring.lean,Mathlib/Order/Filter/AtTopBot/CountablyGenerated.lean,Mathlib/Order/Filter/Cocardinal.lean,Mathlib/Order/Filter/Cofinite.lean,Mathlib/Order/Filter/Tendsto.lean,Mathlib/Order/Filter/Ultrafilter/Basic.lean,Mathlib/Probability/Distributions/Uniform.lean,Mathlib/Probability/Kernel/Basic.lean,Mathlib/Probability/Kernel/Composition/MeasureCompProd.lean,Mathlib/RingTheory/AdicCompletion/LocalRing.lean,Mathlib/RingTheory/Ideal/Maximal.lean,Mathlib/RingTheory/LaurentSeries.lean,Mathlib/RingTheory/MvPolynomial/Symmetric/NewtonIdentities.lean,Mathlib/RingTheory/MvPowerSeries/NoZeroDivisors.lean,Mathlib/RingTheory/Spectrum/Maximal/Localization.lean,Mathlib/RingTheory/Spectrum/Prime/RingHom.lean,Mathlib/RingTheory/Spectrum/Prime/Topology.lean,Mathlib/Topology/Algebra/InfiniteSum/Group.lean,Mathlib/Topology/Algebra/Module/Cardinality.lean,Mathlib/Topology/Algebra/Support.lean,Mathlib/Topology/Bases.lean,Mathlib/Topology/ContinuousMap/BoundedCompactlySupported.lean,Mathlib/Topology/Order/Basic.lean,Mathlib/Topology/UrysohnsLemma.lean 77 4 ['b-mehta', 'github-actions', 'jcommelin', 'leanprover-community-bot-assistant', 'mathlib-bors'] nobody
7-49043
7 days ago
7-49043
7 days ago
0-55045
15 hours
24396 JovanGerb
author:JovanGerb
feat(Order/Defs): refactor in preparation of `to_dual` attribute When the `to_dual` attribute lands in Mathlib, we will tag many lemmas about order with this tag, which will automatically give us the dual statements. This PR prepares for this by - moving dual declarations closer together - replacing occurrences of `>` and `≥` with `<` and `≤` - consistently applying a new naming convention that helps us to name dual lemmas: we use the keywords `ge` and `gt` in place of `le` and `lt` to indicate that the same pair `a, b` in `a < b` is in the opposite order to the order in which it appeared the first time. - when we have to disambiguate the order of the argument to `<` or `≤`, we sometimes use `gt` or `ge` instead of `lt` or `le`. We also use this to get rid of many primed lemma names. This is a copy of #24376, but it doesn't remove the old lemma names, so doesn't require making changes in >500 files. deprecating these lemmas will be left to a future PR. [#mathlib4 > naming convention for ≤ and <](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/naming.20convention.20for.20.E2.89.A4.20and.20.3C) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-zulip t-order merge-conflict 248/230 Mathlib/Algebra/Order/CauSeq/Basic.lean,Mathlib/Algebra/Order/Ring/Unbundled/Rat.lean,Mathlib/Algebra/Polynomial/Degree/Domain.lean,Mathlib/Algebra/Tropical/Basic.lean,Mathlib/Analysis/SpecialFunctions/Pow/Continuity.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Arctan.lean,Mathlib/Computability/TuringMachine.lean,Mathlib/Data/Bool/Basic.lean,Mathlib/Data/Char.lean,Mathlib/Data/Complex/Order.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/Data/Int/Order/Basic.lean,Mathlib/Data/Nat/Basic.lean,Mathlib/Data/Nat/Factorization/Defs.lean,Mathlib/Data/Nat/Find.lean,Mathlib/Data/Nat/PartENat.lean,Mathlib/Data/Num/Lemmas.lean,Mathlib/Data/Num/ZNum.lean,Mathlib/Data/PSigma/Order.lean,Mathlib/Data/Prod/Lex.lean,Mathlib/Data/Real/Basic.lean,Mathlib/Data/Setoid/Basic.lean,Mathlib/Data/Setoid/Partition.lean,Mathlib/Data/Sigma/Order.lean,Mathlib/Data/String/Basic.lean,Mathlib/Data/Sum/Order.lean,Mathlib/GroupTheory/MonoidLocalization/Order.lean,Mathlib/NumberTheory/Zsqrtd/Basic.lean,Mathlib/Order/Antisymmetrization.lean,Mathlib/Order/Basic.lean,Mathlib/Order/Booleanisation.lean,Mathlib/Order/Defs/LinearOrder.lean,Mathlib/Order/Defs/PartialOrder.lean,Mathlib/Order/RelClasses.lean,Mathlib/Order/WithBot.lean,Mathlib/Probability/Martingale/Upcrossing.lean,Mathlib/RingTheory/UniqueFactorizationDomain/Multiplicity.lean,Mathlib/SetTheory/Game/Basic.lean,Mathlib/SetTheory/Ordinal/Basic.lean,Mathlib/SetTheory/Ordinal/Notation.lean,Mathlib/SetTheory/Surreal/Basic.lean,Mathlib/Tactic/Linarith/Frontend.lean,MathlibTest/linarith.lean 43 5 ['JovanGerb', 'bryangingechen', 'github-actions', 'leanprover-community-bot-assistant'] bryangingechen
assignee:bryangingechen
7-11145
7 days ago
7-11147
7 days ago
5-75236
5 days

PRs with just a merge conflict

Number Author Title Description Labels +/- Modified files (first 100) 📝 💬 All users who commented or reviewed Assignee(s) Updated Last status change total time in review
12936 mattrobball
author:mattrobball
chore(Quiver.Opposite): make `Quiver.Hom.op/unop` `abbrev`'s These are wrappers around the constructor and projection for `Opposite Quiver.Hom _ _`. The projection itself is reducible and with structure eta built in to defeq it seems like we might be making Lean work harder than is necessary. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict 39/34 Mathlib/Algebra/Homology/ShortComplex/Homology.lean,Mathlib/Algebra/Homology/ShortComplex/RightHomology.lean,Mathlib/CategoryTheory/Idempotents/Basic.lean,Mathlib/CategoryTheory/Limits/HasLimits.lean,Mathlib/CategoryTheory/Limits/Opposites.lean,Mathlib/CategoryTheory/Opposites.lean,Mathlib/CategoryTheory/Sites/CoverLifting.lean,Mathlib/CategoryTheory/Subobject/Comma.lean,Mathlib/CategoryTheory/Triangulated/Opposite.lean,Mathlib/Combinatorics/Quiver/Basic.lean 10 9 ['YaelDillies', 'kim-em', 'leanprover-bot', 'mattrobball'] nobody
313-42770
10 months ago
381-8762
1 year ago
0-0
0 seconds
10721 urkud
author:urkud
feat(Order/FunLike): define `PointwiseLE` - introduce a mixin class `DFunLike.PointwiseLE`, use it to define `DFunLike.instPartialOrder`; - add a generic `DFunLike.orderEmbeddingCoe` - add `DFunLike.PointwiseLE` instances here and there. With this refactor and #13022, I'm going to generalize lemmas like `MeasureTheory.ae_mono` to `OuterMeasureClass`. --- - [x] depends on: #12983 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-logic t-order merge-conflict 123/50 Mathlib.lean,Mathlib/Algebra/Order/Hom/Ring.lean,Mathlib/Data/DFinsupp/Order.lean,Mathlib/Data/Finsupp/Order.lean,Mathlib/Data/FunLike/Basic.lean,Mathlib/Dynamics/Circle/RotationNumber/TranslationNumber.lean,Mathlib/GroupTheory/Congruence.lean,Mathlib/Order/FunLike.lean,Mathlib/Order/Heyting/Hom.lean,Mathlib/Order/Hom/Basic.lean,Mathlib/Order/Hom/Bounded.lean,Mathlib/Order/Hom/CompleteLattice.lean,Mathlib/Topology/Order/Hom/Basic.lean 13 48 ['YaelDillies', 'dupuisf', 'leanprover-community-mathlib4-bot', 'urkud'] nobody
313-42768
10 months ago
335-23470
11 months ago
64-12826
64 days
8788 FMLJohn
author:FMLJohn
feat(Algebra/Module/GradeZeroModule): if `A` is a graded semiring and `M` is a graded `A`-module, then each grade of `M` is a module over the 0-th grade of `A`. --- - [ ] depends on: #8187 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict
label:t-algebra$
237/4 Mathlib.lean,Mathlib/Algebra/DirectSum/Internal.lean,Mathlib/Algebra/GradedMonoid.lean,Mathlib/Algebra/Module/GradeZeroModule.lean,Mathlib/RingTheory/GradedAlgebra/Basic.lean,Mathlib/RingTheory/GradedAlgebra/Noetherian.lean 6 4 ['FMLJohn', 'github-actions', 'leanprover-community-mathlib4-bot'] nobody
313-42767
10 months ago
347-30669
11 months ago
0-0
0 seconds
9339 FMLJohn
author:FMLJohn
feat (RingTheory/GradedAlgebra/HomogeneousIdeal): given a finitely generated homogeneous ideal of a graded semiring, construct a finite spanning set for the ideal which only contains homogeneous elements --- - [ ] depends on: #8187 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict
label:t-algebra$
402/4 Mathlib.lean,Mathlib/Algebra/DirectSum/Internal.lean,Mathlib/Algebra/GradedMonoid.lean,Mathlib/Algebra/Module/GradeZeroModule.lean,Mathlib/RingTheory/Finiteness.lean,Mathlib/RingTheory/GradedAlgebra/Basic.lean,Mathlib/RingTheory/GradedAlgebra/HomogeneousIdeal.lean,Mathlib/RingTheory/GradedAlgebra/Noetherian.lean 8 11 ['FMLJohn', 'github-actions', 'jjaassoonn', 'leanprover-community-mathlib4-bot'] nobody
313-42767
10 months ago
347-30684
11 months ago
0-0
0 seconds
7875 FR-vdash-bot
author:FR-vdash-bot
chore: make `SMulCommClass A A B` and `SMulCommClass A B B` higher priority --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) slow-typeclass-synthesis t-algebra merge-conflict
label:t-algebra$
54/48 Mathlib/Algebra/Algebra/Basic.lean,Mathlib/Algebra/Algebra/NonUnitalSubalgebra.lean,Mathlib/Algebra/DirectSum/Algebra.lean,Mathlib/Algebra/Group/Action/Defs.lean,Mathlib/Algebra/Group/Subgroup/Actions.lean,Mathlib/Algebra/Lie/NonUnitalNonAssocAlgebra.lean,Mathlib/Algebra/Module/LinearMap/End.lean,Mathlib/Algebra/MonoidAlgebra/Basic.lean,Mathlib/Algebra/MvPolynomial/Basic.lean,Mathlib/Algebra/Ring/CentroidHom.lean,Mathlib/Algebra/Ring/Subring/Basic.lean,Mathlib/Algebra/Ring/Subsemiring/Basic.lean,Mathlib/Algebra/Star/NonUnitalSubalgebra.lean,Mathlib/Analysis/Complex/UnitDisc/Basic.lean,Mathlib/Analysis/NormedSpace/lpSpace.lean,Mathlib/Data/Matrix/Basic.lean,Mathlib/GroupTheory/GroupAction/Prod.lean,Mathlib/GroupTheory/GroupAction/Ring.lean,Mathlib/GroupTheory/GroupAction/SubMulAction.lean,Mathlib/GroupTheory/MonoidLocalization.lean,Mathlib/GroupTheory/Submonoid/Center.lean,Mathlib/LinearAlgebra/PiTensorProduct.lean,Mathlib/RingTheory/Ideal/Quotient.lean,Mathlib/RingTheory/TensorProduct/Basic.lean,Mathlib/Topology/ContinuousFunction/ContinuousMapZero.lean,Mathlib/Topology/ContinuousFunction/StoneWeierstrass.lean,Mathlib/Topology/ContinuousFunction/ZeroAtInfty.lean 27 15 ['FR-vdash-bot', 'Parcly-Taxel', 'jcommelin', 'leanprover-bot'] nobody
313-42766
10 months ago
335-23470
11 months ago
1-47913
1 day
6777 adomani
author:adomani
chore(Co*variantClass): replace eta-expanded (· * ·), (· + ·), (· ≤ ·), (· < ·) Replace `CovariantClass X X (· * ·) (· ≤ ·)` with -> `CovariantClass X X HMul.hMul LE.le` and similarly for `HAdd`, `LT`, `Contravariant`. This PR is inspired by [Issue #6646](https://github.com/leanprover-community/mathlib4/issues/6646) and, more specifically, [this comment](https://github.com/leanprover-community/mathlib4/issues/6646#issuecomment-1692792066). Note that https://github.com/leanprover/lean4/pull/2267 would make this unnecessary --- ```bash # First sed command: # the first captured pattern is `Co*variantClass ` # the second captured pattern is `` # the third captured pattern is `+` or `*` # the fourth captured pattern is `<` or `≤` # a match for `Co*variantClass ·) (· ·)` becomes # `Co*variantClass replaceop replaceop` # Second sed command: similar to the first, but looks for `(Function.swap (· ·))` sed -i ' s=\(Co[ntra]*variantClass \(..*\) \2 \)(· *\([+*]\) *·) (· *\([<≤]\) *·)=\1replaceop\3 replaceop\4=g s=\(Co[ntra]*variantClass \(..*\) \2 \)(\([Functio\.swap ]*\)(· *\([+*]\) *·)) (· *\([<≤]\) *·)=\1(\3replaceop\4) replaceop\5=g s=replaceop+=HAdd.hAdd=g s=replaceop\*=HMul.hMul=g s=replaceop<=LT.lt=g s=replaceop≤=LE.le=g s=\(Co[ntra]*variantClass N N\) (· \* ·) r=\1 HMul.hMul r=g s=\(Co[ntra]*variantClass N N (swap μ)\) (· ≤ ·)=\1 LE.le=g s=\(Co[ntra]*variantClass N N\) (swap (· \* ·)) r=\1 (swap HMul.hMul) r=g s=\(CovariantClass (Filter α) (Filter α)\) (· / ·) (· ≤ ·)=\1 HDiv.hDiv LE.le=g s=\(CovariantClass (Filter α) (Filter α)\) (swap (· / ·)) (· ≤ ·)=\1 (swap HDiv.hDiv) LE.le=g s=\(Co[ntra]*variantClass .* (fun x y .> . \* .)\) (· ≤ ·)=\1 LE.le=g s=\(Co[ntra]*variantClass .* (fun x y .> . \* .)\) (· < ·)=\1 LT.lt=g s=\(Co[ntra]*variantClass [^}]*\) (· ≤ ·)=\1 LE.le=g s=\(CovariantClass .* (Filter β)\) (· • ·) LE.le=\1 HSMul.hSMul LE.le=g ' $(git ls-files '*.lean') ``` [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict 703/678 Counterexamples/ZeroDivisorsInAddMonoidAlgebras.lean,Mathlib/Algebra/BigOperators/Basic.lean,Mathlib/Algebra/Bounds.lean,Mathlib/Algebra/CovariantAndContravariant.lean,Mathlib/Algebra/DirectSum/Internal.lean,Mathlib/Algebra/Group/UniqueProds.lean,Mathlib/Algebra/GroupPower/Order.lean,Mathlib/Algebra/MonoidAlgebra/Degree.lean,Mathlib/Algebra/Order/Archimedean.lean,Mathlib/Algebra/Order/Group/Abs.lean,Mathlib/Algebra/Order/Group/Defs.lean,Mathlib/Algebra/Order/Group/DenselyOrdered.lean,Mathlib/Algebra/Order/Group/MinMax.lean,Mathlib/Algebra/Order/Group/OrderIso.lean,Mathlib/Algebra/Order/Hom/Monoid.lean,Mathlib/Algebra/Order/Interval.lean,Mathlib/Algebra/Order/Kleene.lean,Mathlib/Algebra/Order/LatticeGroup.lean,Mathlib/Algebra/Order/Module.lean,Mathlib/Algebra/Order/Monoid/Basic.lean,Mathlib/Algebra/Order/Monoid/Cancel/Defs.lean,Mathlib/Algebra/Order/Monoid/Canonical/Defs.lean,Mathlib/Algebra/Order/Monoid/Defs.lean,Mathlib/Algebra/Order/Monoid/Lemmas.lean,Mathlib/Algebra/Order/Monoid/MinMax.lean,Mathlib/Algebra/Order/Monoid/NatCast.lean,Mathlib/Algebra/Order/Monoid/OrderDual.lean,Mathlib/Algebra/Order/Monoid/Prod.lean,Mathlib/Algebra/Order/Monoid/WithTop.lean,Mathlib/Algebra/Order/Monoid/WithZero/Basic.lean,Mathlib/Algebra/Order/Monoid/WithZero/Defs.lean,Mathlib/Algebra/Order/Nonneg/Ring.lean,Mathlib/Algebra/Order/Pointwise.lean,Mathlib/Algebra/Order/Positive/Ring.lean,Mathlib/Algebra/Order/Ring/Canonical.lean,Mathlib/Algebra/Order/Ring/Defs.lean,Mathlib/Algebra/Order/Ring/Lemmas.lean,Mathlib/Algebra/Order/Sub/Basic.lean,Mathlib/Algebra/Order/Sub/Canonical.lean,Mathlib/Algebra/Order/Sub/Defs.lean,Mathlib/Algebra/Order/WithZero.lean,Mathlib/Algebra/Parity.lean,Mathlib/Algebra/Star/Order.lean,Mathlib/Algebra/Tropical/Basic.lean,Mathlib/Analysis/Normed/Order/Lattice.lean,Mathlib/Data/DFinsupp/Lex.lean,Mathlib/Data/DFinsupp/Order.lean,Mathlib/Data/Finset/Fold.lean,Mathlib/Data/Finsupp/Lex.lean,Mathlib/Data/Finsupp/Order.lean,Mathlib/Data/List/BigOperators/Basic.lean,Mathlib/Data/List/BigOperators/Lemmas.lean,Mathlib/Data/Multiset/Basic.lean,Mathlib/Data/Nat/Cast/Order.lean,Mathlib/Data/PNat/Basic.lean,Mathlib/Data/Real/ENNReal.lean,Mathlib/Data/Real/NNReal.lean,Mathlib/Data/Set/Semiring.lean,Mathlib/Data/Sign.lean,Mathlib/MeasureTheory/Function/LpOrder.lean,Mathlib/MeasureTheory/Function/SimpleFuncDenseLp.lean,Mathlib/MeasureTheory/Measure/MeasureSpace.lean,Mathlib/MeasureTheory/Measure/VectorMeasure.lean,Mathlib/Order/ConditionallyCompleteLattice/Group.lean,Mathlib/Order/Filter/Basic.lean,Mathlib/Order/Filter/Pointwise.lean,Mathlib/Probability/Martingale/Basic.lean,Mathlib/Probability/Process/Stopping.lean,Mathlib/RingTheory/GradedAlgebra/Basic.lean,Mathlib/SetTheory/Cardinal/Basic.lean,Mathlib/SetTheory/Game/Basic.lean,Mathlib/SetTheory/Game/PGame.lean,Mathlib/SetTheory/Ordinal/Arithmetic.lean,Mathlib/SetTheory/Ordinal/Basic.lean,Mathlib/SetTheory/Ordinal/NaturalOps.lean,Mathlib/Tactic/GCongr/Core.lean,Mathlib/Tactic/Positivity/Basic.lean,Mathlib/Topology/ContinuousFunction/Algebra.lean,lean-toolchain,test/Recall.lean,test/propose.lean 81 36 ['adomani', 'alreadydone', 'digama0', 'eric-wieser', 'ericrbg', 'jcommelin', 'leanprover-bot', 'sgouezel'] nobody
313-42766
10 months ago
335-23470
11 months ago
35-56459
35 days
6993 jjaassoonn
author:jjaassoonn
feat : lemmas about `AddMonoidAlgebra.{divOf, modOf}` --- - [x] depends on: #7582 - [x] depends on: #8975 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict
label:t-algebra$
147/3 Mathlib/Algebra/MonoidAlgebra/Division.lean,Mathlib/Data/Finsupp/Basic.lean,Mathlib/Data/MvPolynomial/Basic.lean,Mathlib/Data/MvPolynomial/CommRing.lean,Mathlib/Data/MvPolynomial/Division.lean 5 42 ['YaelDillies', 'alreadydone', 'digama0', 'eric-wieser', 'github-actions', 'jjaassoonn', 'leanprover-community-mathlib4-bot'] nobody
313-42765
10 months ago
335-23470
11 months ago
102-21189
102 days
6491 eric-wieser
author:eric-wieser
chore(Mathlib/Algebra/Hom/GroupAction): add `SMulHomClass.comp_smul` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict
label:t-algebra$
24/10 Mathlib/Algebra/Hom/GroupAction.lean 1 0 [] nobody
313-42765
10 months ago
335-23470
11 months ago
83-76369
83 days
10629 madvorak
author:madvorak
feat: List.cons_sublist_append_iff_right --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data merge-conflict 11/0 Mathlib/Data/List/Basic.lean 1 1 ['eric-wieser'] nobody
299-36310
9 months ago
299-36310
9 months ago
53-73442
53 days
11632 mattrobball
author:mattrobball
chore(Group/RingTheory.Congruence): make `Quotient`'s reducible These are essentially wrappers and should not expose any data when made reducible. Their use in constructing typeclass instances makes reducible transparency desirable. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict 16/35 Mathlib/GroupTheory/Congruence/Basic.lean,Mathlib/RingTheory/Congruence/Basic.lean 2 14 ['eric-wieser', 'fpvandoorn', 'github-actions', 'grunweg', 'kmill', 'leanprover-bot', 'mattrobball'] nobody
294-85734
9 months ago
325-21094
10 months ago
2-10495
2 days
13791 digama0
author:digama0
refactor: Primrec and Partrec General cleanup of the `Primrec` and `Partrec` files, to better adjust to lean 4 things. The main user-visible change is that `Primrec₂` is no longer a `def` but an `abbrev`, because it was causing inference issues in lean 4. I also removed all the nonterminal `simp`s in `PartrecCode.lean`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) tech debt t-computability merge-conflict 585/778 Mathlib/Computability/Ackermann.lean,Mathlib/Computability/Halting.lean,Mathlib/Computability/Partrec.lean,Mathlib/Computability/PartrecCode.lean,Mathlib/Computability/Primrec.lean 5 2 ['github-actions', 'grunweg'] nobody
294-85555
9 months ago
335-23470
11 months ago
1-84718
1 day
11964 adamtopaz
author:adamtopaz
feat: The functor of points of a scheme We construct the functor of points functor, and prove that it's full and faithful. --- - [ ] depends on: #11947 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebraic-geometry t-category-theory merge-conflict 210/0 Mathlib.lean,Mathlib/AlgebraicGeometry/FunctorOfPoints.lean,Mathlib/AlgebraicGeometry/OpenImmersion.lean 3 4 ['github-actions', 'grunweg', 'leanprover-community-mathlib4-bot'] nobody
294-85414
9 months ago
335-23470
11 months ago
0-1223
20 minutes
12418 rosborn
author:rosborn
style: replace preimage_val with ↓∩ notation --- This is a rough draft of what the new `↓∩` notation would look like within mathlib. I believe this is an improvement in clarity and would like to have `↓∩` as a standard notation (along with `''`, `⁻¹'`, `↑`, etc...). As `↓∩` is specialized for `Set`s, I have only changed `preimage_val` when the left-hand side of `↓∩` is a `Set`. The introduction of the `↓∩` notation to Data.Set.Image is temporary as it isn't possible to import Data.Set.Subset directly. If we want `↓∩` unscoped, where would be the best place to define it? An option is Data.Set.Defs, but the notation cannot be defined without additional imports as the file does not import `notation3`. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict 56/61 Mathlib/Analysis/InnerProductSpace/Projection.lean,Mathlib/Data/Set/Function.lean,Mathlib/Data/Set/Image.lean,Mathlib/Data/Set/Subset.lean,Mathlib/MeasureTheory/Constructions/Polish.lean,Mathlib/MeasureTheory/MeasurableSpace/Basic.lean,Mathlib/MeasureTheory/Measure/Restrict.lean,Mathlib/Order/UpperLower/Basic.lean,Mathlib/Topology/Bases.lean,Mathlib/Topology/Clopen.lean,Mathlib/Topology/Connected/Basic.lean,Mathlib/Topology/Connected/PathConnected.lean,Mathlib/Topology/Constructions.lean,Mathlib/Topology/ContinuousOn.lean,Mathlib/Topology/LocalAtTarget.lean,Mathlib/Topology/LocallyConstant/Basic.lean,Mathlib/Topology/Separation.lean,Mathlib/Topology/Sober.lean 18 3 ['grunweg', 'rosborn'] nobody
294-85313
9 months ago
335-23470
11 months ago
29-14218
29 days
12751 Command-Master
author:Command-Master
feat: add lemmas for Nat/Bits, Nat/Bitwise and Nat/Size Remove `@[simp]` from `Nat.bit_false` and `Nat.bit_true`, as `bit0` and `bit1` are deprecated, and add some lemmas to `Bits`, `Bitwise` and `Size`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data new-contributor merge-conflict 66/7 Mathlib/Data/Nat/Bits.lean,Mathlib/Data/Nat/Bitwise.lean,Mathlib/Data/Nat/Multiplicity.lean,Mathlib/Data/Nat/Size.lean 4 26 ['Command-Master', 'Rida-Hamadani', 'Ruben-VandeVelde', 'YaelDillies', 'github-actions', 'jcommelin'] nobody
294-20067
9 months ago
299-36309
9 months ago
54-52408
54 days
16464 Parcly-Taxel
author:Parcly-Taxel
chore: deprecate `Nat.(case_)strong_induction_on` …in favour of the now-renamed `Nat.(case)strongInductionOn` in core. tech debt merge-conflict 54/56 Archive/Imo/Imo1981Q3.lean,Mathlib/Algebra/ContinuedFractions/Computation/Approximations.lean,Mathlib/Algebra/ContinuedFractions/Computation/TerminatesIffRat.lean,Mathlib/Algebra/ContinuedFractions/ConvergentsEquiv.lean,Mathlib/Algebra/Polynomial/Derivative.lean,Mathlib/Algebra/Polynomial/Lifts.lean,Mathlib/Analysis/Analytic/Basic.lean,Mathlib/Analysis/Calculus/ContDiff/Bounds.lean,Mathlib/Analysis/Hofer.lean,Mathlib/Analysis/SpecificLimits/Normed.lean,Mathlib/Combinatorics/Derangements/Finite.lean,Mathlib/Combinatorics/Enumerative/Catalan.lean,Mathlib/Combinatorics/Hall/Finite.lean,Mathlib/Combinatorics/SetFamily/AhlswedeZhang.lean,Mathlib/Computability/Primrec.lean,Mathlib/Data/Fintype/Basic.lean,Mathlib/Data/Fintype/Card.lean,Mathlib/Data/Nat/Choose/Central.lean,Mathlib/Data/Nat/Defs.lean,Mathlib/Data/Nat/Digits.lean,Mathlib/Data/Nat/Log.lean,Mathlib/FieldTheory/Separable.lean,Mathlib/LinearAlgebra/Eigenspace/Triangularizable.lean,Mathlib/LinearAlgebra/Multilinear/Basic.lean,Mathlib/NumberTheory/BernoulliPolynomials.lean,Mathlib/NumberTheory/DiophantineApproximation.lean,Mathlib/NumberTheory/Pell.lean,Mathlib/NumberTheory/Primorial.lean,Mathlib/Order/Fin/Basic.lean,Mathlib/RingTheory/Adjoin/PowerBasis.lean,Mathlib/RingTheory/LittleWedderburn.lean,Mathlib/RingTheory/Polynomial/Basic.lean,Mathlib/RingTheory/Polynomial/Cyclotomic/Basic.lean,Mathlib/RingTheory/Polynomial/Cyclotomic/Eval.lean,Mathlib/RingTheory/Polynomial/Eisenstein/IsIntegral.lean,Mathlib/RingTheory/Polynomial/Nilpotent.lean,Mathlib/RingTheory/PowerSeries/Basic.lean,Mathlib/RingTheory/QuotientNilpotent.lean,Mathlib/RingTheory/WittVector/Defs.lean,Mathlib/RingTheory/WittVector/Frobenius.lean,Mathlib/RingTheory/WittVector/StructurePolynomial.lean,Mathlib/SetTheory/Surreal/Dyadic.lean,Mathlib/Topology/Metrizable/Uniformity.lean 43 13 ['Parcly-Taxel', 'b-mehta', 'github-actions', 'jcommelin'] nobody
262-8623
8 months ago
262-8623
8 months ago
8-1989
8 days
17127 FR-vdash-bot
author:FR-vdash-bot
chore: remove global `Quotient.mk` `⟦·⟧` notation --- Merge this PR when we are ready to migrate to `QuotLike` API (#16421). [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data merge-conflict 137/2 Counterexamples/Pseudoelement.lean,Mathlib/Algebra/Associated/Basic.lean,Mathlib/Algebra/BigOperators/Group/Finset.lean,Mathlib/Algebra/Group/Conj.lean,Mathlib/Algebra/GroupWithZero/NonZeroDivisors.lean,Mathlib/Algebra/Order/CauSeq/Completion.lean,Mathlib/Algebra/Quandle.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Jacobian.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Projective.lean,Mathlib/AlgebraicTopology/FundamentalGroupoid/Basic.lean,Mathlib/AlgebraicTopology/FundamentalGroupoid/FundamentalGroup.lean,Mathlib/AlgebraicTopology/FundamentalGroupoid/InducedMaps.lean,Mathlib/AlgebraicTopology/FundamentalGroupoid/Product.lean,Mathlib/AlgebraicTopology/FundamentalGroupoid/SimplyConnected.lean,Mathlib/CategoryTheory/Abelian/Pseudoelements.lean,Mathlib/CategoryTheory/Limits/Shapes/SingleObj.lean,Mathlib/CategoryTheory/Monoidal/Free/Basic.lean,Mathlib/CategoryTheory/Monoidal/Free/Coherence.lean,Mathlib/CategoryTheory/Skeletal.lean,Mathlib/Data/Finset/Card.lean,Mathlib/Data/Fintype/List.lean,Mathlib/Data/Fintype/Quotient.lean,Mathlib/Data/Multiset/Basic.lean,Mathlib/Data/QPF/Multivariate/Constructions/Fix.lean,Mathlib/Data/QPF/Univariate/Basic.lean,Mathlib/Data/Quot.lean,Mathlib/Data/Real/Basic.lean,Mathlib/Data/Set/Finite.lean,Mathlib/Data/Set/Image.lean,Mathlib/Data/Setoid/Basic.lean,Mathlib/GroupTheory/GroupAction/Basic.lean,Mathlib/GroupTheory/GroupAction/Quotient.lean,Mathlib/LinearAlgebra/Dual.lean,Mathlib/LinearAlgebra/Ray.lean,Mathlib/Logic/Encodable/Basic.lean,Mathlib/Logic/Equiv/Basic.lean,Mathlib/ModelTheory/DirectLimit.lean,Mathlib/ModelTheory/Fraisse.lean,Mathlib/ModelTheory/Quotients.lean,Mathlib/NumberTheory/NumberField/CanonicalEmbedding/FundamentalCone.lean,Mathlib/NumberTheory/NumberField/Embeddings.lean,Mathlib/NumberTheory/NumberField/Units/DirichletTheorem.lean,Mathlib/NumberTheory/Padics/PadicIntegers.lean,Mathlib/NumberTheory/Padics/PadicNumbers.lean,Mathlib/Order/RelIso/Basic.lean,Mathlib/RepresentationTheory/Action/Concrete.lean,Mathlib/SetTheory/Cardinal/Basic.lean,Mathlib/SetTheory/Cardinal/Ordinal.lean,Mathlib/SetTheory/Game/Basic.lean,Mathlib/SetTheory/Game/Birthday.lean,Mathlib/SetTheory/Game/Impartial.lean,Mathlib/SetTheory/Game/Ordinal.lean,Mathlib/SetTheory/Game/State.lean,Mathlib/SetTheory/Lists.lean,Mathlib/SetTheory/Ordinal/Arithmetic.lean,Mathlib/SetTheory/Ordinal/Basic.lean,Mathlib/SetTheory/Surreal/Basic.lean,Mathlib/SetTheory/Surreal/Dyadic.lean,Mathlib/SetTheory/Surreal/Multiplication.lean,Mathlib/SetTheory/ZFC/Basic.lean,Mathlib/SetTheory/ZFC/Rank.lean,Mathlib/Topology/Connected/PathConnected.lean,Mathlib/Topology/Homotopy/HomotopyGroup.lean,Mathlib/Topology/Homotopy/Path.lean,Mathlib/Topology/Homotopy/Product.lean,Mathlib/Topology/MetricSpace/GromovHausdorff.lean,Mathlib/Topology/UniformSpace/Separation.lean,test/interactiveUnfold.lean 68 1 ['github-actions'] nobody
252-57406
8 months ago
252-57406
8 months ago
4-72805
4 days
8029 alreadydone
author:alreadydone
refactor: Homotopy between Functions not ContinuousMaps This allows talking about homotopies without needing to supply proofs of continuity for the two ends. This for example simplifies the definition of H-spaces. Of course, if a homotopy exists between two functions, those two functions are automatically continuous because they are restrictions of the homotopy (which is continuous) to subspaces. `Homotopy.refl` still needs a continuous map as input, and `Homotopic` is only an equivalence relation when restricted to ContinuousMap. --- TODO: fix docstrings [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology RFC merge-conflict 246/250 Mathlib/AlgebraicTopology/FundamentalGroupoid/InducedMaps.lean,Mathlib/Topology/Homotopy/Basic.lean,Mathlib/Topology/Homotopy/Contractible.lean,Mathlib/Topology/Homotopy/Equiv.lean,Mathlib/Topology/Homotopy/HSpaces.lean,Mathlib/Topology/Homotopy/HomotopyGroup.lean,Mathlib/Topology/Homotopy/Path.lean,Mathlib/Topology/Homotopy/Product.lean 8 3 ['alreadydone', 'urkud'] nobody
242-86211
7 months ago
335-23470
11 months ago
9-20043
9 days
14598 Command-Master
author:Command-Master
chore: add typeclasses to unify various `add_top`, `add_eq_top`, etc. Add the four typeclasses `IsTopAbsorbing`, `IsBotAbsorbing`, `NoTopSum`, `NoBotSum`, as additive equivalents for `MulZeroClass` and `NoZeroDivisors`. Add instances of these for `ENNReal`, `WithTop α`, `WithBot α`, `PUnit`, `EReal`, `PartENat`, `Measure`, `Interval` and `Filter`. Also split `Algebra/Order/AddGroupWithTop` to `Algebra/Order/Group/WithTop` and `Algebra/Order/Monoid/WithTop` --- Previous usages of lemmas with quantified names like `WithTop.add_top` have to be changed to just `add_top`. `add_lt_top` is `@[simp]`, in accordance with `ENNReal.add_lt_top` being `@[simp]`. This affects `WithTop.add_lt_top` which previously hadn't been `@[simp]`. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-order t-algebra merge-conflict
label:t-algebra$
264/195 Archive/Wiedijk100Theorems/BallotProblem.lean,Mathlib.lean,Mathlib/Algebra/Order/Group/WithTop.lean,Mathlib/Algebra/Order/GroupWithZero/Canonical.lean,Mathlib/Algebra/Order/Interval/Basic.lean,Mathlib/Algebra/Order/Monoid/Unbundled/Basic.lean,Mathlib/Algebra/Order/Monoid/Unbundled/Defs.lean,Mathlib/Algebra/Order/Monoid/Unbundled/WithTop.lean,Mathlib/Algebra/Order/Monoid/WithTop.lean,Mathlib/Algebra/PUnitInstances/Order.lean,Mathlib/Algebra/Polynomial/Degree/Definitions.lean,Mathlib/Algebra/Polynomial/Monic.lean,Mathlib/Algebra/Tropical/Basic.lean,Mathlib/Analysis/Analytic/Meromorphic.lean,Mathlib/Analysis/Normed/Lp/ProdLp.lean,Mathlib/Analysis/NormedSpace/ENorm.lean,Mathlib/Analysis/SpecialFunctions/JapaneseBracket.lean,Mathlib/Analysis/SpecialFunctions/Log/ENNRealLog.lean,Mathlib/Data/ENNReal/Operations.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/Data/Nat/PartENat.lean,Mathlib/Data/Nat/WithBot.lean,Mathlib/Data/Real/EReal.lean,Mathlib/LinearAlgebra/Lagrange.lean,Mathlib/MeasureTheory/Covering/Differentiation.lean,Mathlib/MeasureTheory/Decomposition/Lebesgue.lean,Mathlib/MeasureTheory/Function/ConditionalExpectation/CondexpL1.lean,Mathlib/MeasureTheory/Function/Jacobian.lean,Mathlib/MeasureTheory/Function/L1Space.lean,Mathlib/MeasureTheory/Function/L2Space.lean,Mathlib/MeasureTheory/Function/LpSeminorm/Basic.lean,Mathlib/MeasureTheory/Function/LpSeminorm/TriangleInequality.lean,Mathlib/MeasureTheory/Function/LpSpace.lean,Mathlib/MeasureTheory/Function/StronglyMeasurable/Basic.lean,Mathlib/MeasureTheory/Function/UniformIntegrable.lean,Mathlib/MeasureTheory/Integral/Bochner.lean,Mathlib/MeasureTheory/Integral/MeanInequalities.lean,Mathlib/MeasureTheory/Integral/SetIntegral.lean,Mathlib/MeasureTheory/Integral/VitaliCaratheodory.lean,Mathlib/MeasureTheory/Measure/Hausdorff.lean,Mathlib/MeasureTheory/Measure/Lebesgue/Basic.lean,Mathlib/MeasureTheory/Measure/LevyProkhorovMetric.lean,Mathlib/MeasureTheory/Measure/MeasureSpace.lean,Mathlib/MeasureTheory/Measure/MeasureSpaceDef.lean,Mathlib/MeasureTheory/Measure/Regular.lean,Mathlib/MeasureTheory/Measure/Typeclasses.lean,Mathlib/NumberTheory/Padics/PadicNumbers.lean,Mathlib/Order/Filter/Pointwise.lean,Mathlib/Probability/Kernel/Defs.lean,Mathlib/Probability/Martingale/Convergence.lean,Mathlib/RingTheory/Multiplicity.lean,Mathlib/RingTheory/MvPowerSeries/NoZeroDivisors.lean,Mathlib/RingTheory/UniqueFactorizationDomain.lean,Mathlib/Topology/EMetricSpace/Defs.lean,Mathlib/Topology/MetricSpace/Bounded.lean,Mathlib/Topology/MetricSpace/HausdorffDistance.lean,Mathlib/Topology/MetricSpace/Lipschitz.lean 57 30 ['Command-Master', 'YaelDillies', 'github-actions'] nobody
215-52872
7 months ago
215-52872
7 months ago
7-45599
7 days
12778 MichaelStollBayreuth
author:MichaelStollBayreuth
perf: decouple algebraic and order hierarchies in type class search Based on the experience gained with [#12680](https://github.com/leanprover-community/mathlib4/pull/12680), this attempts to decouple the algebraic and order hierarchies in type class search. * We lower the priorities of instances like `OrderedSemiring.toSemiring` (which are generated by the `extends` clause with default priority 1000) to 50. * Additionally, we make the default priority available via `open scoped AlgebraOrderInstances` and use that where appropriate. **Motivation:** Looking at instance synthesization traces, it appears that when (e.g.) presented with the goal to find a `Semiring` instance, the algorithm frequently goes down a rabbit hole trying and failing to find order instances. This seems to be caused by the presence of instances like `OrderedSemiring.toSemiring` with default priority, which are tried early in the search, but lead nowhere (after a fairly long time). These instances are created by declarations of the form ```lean class OrderedSemiring (α : Type u) extends Semiring α, OrderedAddCommMonoid α where ... ``` which automatically sets up (among other things) an instance `OrderedSemiring.toSemiring` with default piority. It appears that these instances cannot be removed completely (only locally in a module), so the next best solution is to make them low priority (which is possible also for downstream modules). To provide for situations where these instances are desired, we put a default priority version in the scope `AlgebraOrderInstances`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) slow-typeclass-synthesis t-order t-algebra merge-conflict
label:t-algebra$
306/27 Mathlib/Algebra/Algebra/Subalgebra/Order.lean,Mathlib/Algebra/ContinuedFractions/Computation/ApproximationCorollaries.lean,Mathlib/Algebra/ContinuedFractions/Computation/Approximations.lean,Mathlib/Algebra/Module/Rat.lean,Mathlib/Algebra/Module/Submodule/Order.lean,Mathlib/Algebra/Order/AbsoluteValue.lean,Mathlib/Algebra/Order/Algebra.lean,Mathlib/Algebra/Order/Antidiag/Prod.lean,Mathlib/Algebra/Order/Archimedean/Basic.lean,Mathlib/Algebra/Order/BigOperators/Group/Finset.lean,Mathlib/Algebra/Order/BigOperators/Group/List.lean,Mathlib/Algebra/Order/BigOperators/Group/Multiset.lean,Mathlib/Algebra/Order/BigOperators/Ring/Finset.lean,Mathlib/Algebra/Order/BigOperators/Ring/List.lean,Mathlib/Algebra/Order/BigOperators/Ring/Multiset.lean,Mathlib/Algebra/Order/CauSeq/Basic.lean,Mathlib/Algebra/Order/Chebyshev.lean,Mathlib/Algebra/Order/CompleteField.lean,Mathlib/Algebra/Order/Field/Basic.lean,Mathlib/Algebra/Order/Field/Defs.lean,Mathlib/Algebra/Order/Field/Pi.lean,Mathlib/Algebra/Order/Floor.lean,Mathlib/Algebra/Order/Floor/Div.lean,Mathlib/Algebra/Order/Group/Defs.lean,Mathlib/Algebra/Order/Group/Units.lean,Mathlib/Algebra/Order/GroupWithZero/Canonical.lean,Mathlib/Algebra/Order/Hom/Basic.lean,Mathlib/Algebra/Order/Hom/Monoid.lean,Mathlib/Algebra/Order/Interval/Basic.lean,Mathlib/Algebra/Order/Interval/Set/Instances.lean,Mathlib/Algebra/Order/Invertible.lean,Mathlib/Algebra/Order/Kleene.lean,Mathlib/Algebra/Order/Module/Algebra.lean,Mathlib/Algebra/Order/Module/Defs.lean,Mathlib/Algebra/Order/Module/Pointwise.lean,Mathlib/Algebra/Order/Monoid/Basic.lean,Mathlib/Algebra/Order/Monoid/Canonical/Defs.lean,Mathlib/Algebra/Order/Monoid/Defs.lean,Mathlib/Algebra/Order/Monoid/OrderDual.lean,Mathlib/Algebra/Order/Monoid/Prod.lean,Mathlib/Algebra/Order/Nonneg/Field.lean,Mathlib/Algebra/Order/Nonneg/Ring.lean,Mathlib/Algebra/Order/Pi.lean,Mathlib/Algebra/Order/Positive/Field.lean,Mathlib/Algebra/Order/Positive/Ring.lean,Mathlib/Algebra/Order/Rearrangement.lean,Mathlib/Algebra/Order/Ring/Basic.lean,Mathlib/Algebra/Order/Ring/Defs.lean,Mathlib/Algebra/Order/Ring/InjSurj.lean,Mathlib/Algebra/Order/Ring/Pow.lean,Mathlib/Algebra/Order/Sub/WithTop.lean,Mathlib/Algebra/Order/ToIntervalMod.lean,Mathlib/Algebra/Ring/BooleanRing.lean,Mathlib/AlgebraicGeometry/Morphisms/RingHomProperties.lean,Mathlib/AlgebraicTopology/FundamentalGroupoid/Basic.lean,Mathlib/Analysis/BoundedVariation.lean,Mathlib/Analysis/Complex/UpperHalfPlane/Metric.lean,Mathlib/Analysis/Convex/Basic.lean,Mathlib/Analysis/Convex/Cone/Basic.lean,Mathlib/Analysis/Convex/Cone/Closure.lean,Mathlib/Analysis/Convex/Cone/Pointed.lean,Mathlib/Analysis/Convex/Cone/Proper.lean,Mathlib/Analysis/Convex/Exposed.lean,Mathlib/Analysis/Convex/Extrema.lean,Mathlib/Analysis/Convex/Function.lean,Mathlib/Analysis/Convex/Gauge.lean,Mathlib/Analysis/Convex/GaugeRescale.lean,Mathlib/Analysis/Convex/Hull.lean,Mathlib/Analysis/Convex/Join.lean,Mathlib/Analysis/Convex/Mul.lean,Mathlib/Analysis/Convex/Quasiconvex.lean,Mathlib/Analysis/Convex/SpecificFunctions/Pow.lean,Mathlib/Analysis/Convex/Star.lean,Mathlib/Analysis/Convex/Strict.lean,Mathlib/Analysis/InnerProductSpace/Orientation.lean,Mathlib/Analysis/MeanInequalities.lean,Mathlib/Analysis/SpecialFunctions/Gamma/BohrMollerup.lean,Mathlib/Analysis/SpecialFunctions/Polynomials.lean,Mathlib/Analysis/SpecificLimits/FloorPow.lean,Mathlib/Analysis/SpecificLimits/Normed.lean,Mathlib/Combinatorics/Optimization/ValuedCSP.lean,Mathlib/Combinatorics/Pigeonhole.lean,Mathlib/Combinatorics/SetFamily/FourFunctions.lean,Mathlib/Data/DFinsupp/Lex.lean,Mathlib/Data/DFinsupp/Multiset.lean,Mathlib/Data/DFinsupp/Order.lean,Mathlib/Data/Finset/MulAntidiagonal.lean,Mathlib/Data/Finsupp/Lex.lean,Mathlib/Data/Finsupp/Multiset.lean,Mathlib/Data/Finsupp/Order.lean,Mathlib/Data/Int/Log.lean,Mathlib/Data/Multiset/Antidiagonal.lean,Mathlib/Data/Multiset/Basic.lean,Mathlib/Data/Multiset/Bind.lean,Mathlib/Data/Nat/Cast/Field.lean,Mathlib/Data/Nat/Cast/Order/Basic.lean,Mathlib/Data/Nat/Choose/Bounds.lean,Mathlib/Data/PNat/Factors.lean,Mathlib/Data/Rat/Denumerable.lean,Mathlib/Data/Set/Pointwise/Interval.lean 135 34 ['MichaelStollBayreuth', 'YaelDillies', 'github-actions', 'leanprover-bot'] nobody
215-51775
7 months ago
215-51775
7 months ago
18-19513
18 days
18806 FR-vdash-bot
author:FR-vdash-bot
refactor: deprecate `MulEquivClass` --- - [x] depends on: #18809 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict
label:t-algebra$
84/72 Mathlib/Algebra/Group/Equiv/Basic.lean,Mathlib/Algebra/Group/Units/Equiv.lean,Mathlib/Algebra/GroupWithZero/Hom.lean,Mathlib/Algebra/GroupWithZero/NonZeroDivisors.lean,Mathlib/Algebra/Module/Equiv/Defs.lean,Mathlib/Algebra/Order/Hom/Monoid.lean,Mathlib/Algebra/Prime/Lemmas.lean,Mathlib/Algebra/Ring/Divisibility/Basic.lean,Mathlib/Algebra/Ring/Equiv.lean,Mathlib/Combinatorics/Additive/FreimanHom.lean,Mathlib/RingTheory/Bialgebra/Equiv.lean,Mathlib/RingTheory/Ideal/Norm.lean,Mathlib/RingTheory/Localization/FractionRing.lean,Mathlib/RingTheory/Multiplicity.lean,Mathlib/Topology/Algebra/InfiniteSum/Basic.lean 15 6 ['FR-vdash-bot', 'github-actions', 'leanprover-bot', 'mathlib4-dependent-issues-bot', 'vihdzp'] nobody
203-9053
6 months ago
203-9053
6 months ago
4-31794
4 days
19212 Julian
author:Julian
feat(LinearAlgebra): add a variable_alias for VectorSpace Taken directly from the variable_alias docs. Zulip: https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/why.20.5Bvariable_alias.5D.20attribute.20is.20not.20used.20in.20Mathlib.3F --- This is the first actual variable alias added to mathlib. I haven't reviewed variable_alias fully, but it seems like there's at least 3 ways they could be distributed in Mathlib: * alongside whatever subfolder they "belong to" (which is what I've tentatively done here) * In a file called `Aliases` somewhere near the thing they alias (which seems less discoverable to me) * In a single file, a la `Mathlib.TrainingWheels` (with some less playful name) which is meant to define a bunch of more "friendly" aliases all in one place. I kind of like the idea of the third thing as a future module but perhaps it can be synthesized if/when there are more aliases? For now as I say I've done the first one, but please let me know if someone prefers something else. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict
label:t-algebra$
25/0 Mathlib.lean,Mathlib/LinearAlgebra/VectorSpace.lean,scripts/noshake.json 3 10 ['Julian', 'PieterCuijpers', 'github-actions', 'urkud'] nobody
195-29627
6 months ago
195-29627
6 months ago
7-68492
7 days
19337 zeramorphic
author:zeramorphic
feat(Data/Finsupp): generalise `Finsupp` to any "zero" value Remove the explicit dependence of `Finsupp` on `[Zero M]`, instead defining `Finsupp'` (better name pending) to be functions that are equal to a fixed value `z : M` cofinitely often. This PR is intended to do the initial work of replacing the definition of `Finsupp` with an instantiation of the more general definition, without adding any appropriate API. If accepted, the API development will follow in later PRs. Issues to consider: - Naming of `Finsupp'.` - Where should `Finsupp'` lemmas go? Do they need their own file/folder under `Data/`? Relevant Zulip threads: - https://leanprover.zulipchat.com/#narrow/channel/217875-Is-there-code-for-X.3F/topic/Finsupp.20generalisations - https://leanprover.zulipchat.com/#narrow/channel/217875-Is-there-code-for-X.3F/topic/Finsupp-like.20partial.20function Comments are welcome. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data merge-conflict 203/83 Archive/Wiedijk100Theorems/Partition.lean,Mathlib/Algebra/MvPolynomial/Basic.lean,Mathlib/Algebra/MvPolynomial/Rename.lean,Mathlib/Algebra/MvPolynomial/Variables.lean,Mathlib/Algebra/Polynomial/Basic.lean,Mathlib/Algebra/Polynomial/Laurent.lean,Mathlib/Data/Finsupp/BigOperators.lean,Mathlib/Data/Finsupp/Defs.lean,Mathlib/Data/Finsupp/Order.lean,Mathlib/Data/Nat/Choose/Multinomial.lean,Mathlib/RingTheory/MvPolynomial/Symmetric/Defs.lean,Mathlib/RingTheory/PowerBasis.lean,scripts/nolints_prime_decls.txt 13 5 ['github-actions', 'vihdzp', 'zeramorphic'] nobody
193-5704
6 months ago
193-5704
6 months ago
4-60621
4 days
18756 FR-vdash-bot
author:FR-vdash-bot
refactor: deprecate `DistribMulActionSemiHomClass` `MulSemiringActionSemiHomClass` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict
label:t-algebra$
50/28 Mathlib/Algebra/Algebra/NonUnitalHom.lean,Mathlib/Algebra/Module/LinearMap/Defs.lean,Mathlib/GroupTheory/GroupAction/Hom.lean 3 4 ['FR-vdash-bot', 'github-actions', 'leanprover-bot'] nobody
181-57773
5 months ago
181-57773
5 months ago
31-75259
31 days
19046 j-loreaux
author:j-loreaux
feat: define class `SemigroupAction` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict
label:t-algebra$
34/25 Mathlib/Algebra/Category/ModuleCat/Presheaf.lean,Mathlib/Algebra/Category/ModuleCat/Presheaf/Pushforward.lean,Mathlib/Algebra/Group/Action/Defs.lean,Mathlib/Algebra/Group/Action/End.lean,Mathlib/Algebra/Group/Action/Prod.lean,Mathlib/Algebra/Group/Action/TypeTags.lean,Mathlib/Algebra/Polynomial/Laurent.lean,Mathlib/Analysis/Distribution/SchwartzSpace.lean,Mathlib/GroupTheory/CoprodI.lean,Mathlib/LinearAlgebra/FreeModule/IdealQuotient.lean,Mathlib/LinearAlgebra/Matrix/SesquilinearForm.lean 11 7 ['alreadydone', 'github-actions', 'j-loreaux', 'leanprover-bot', 'urkud'] nobody
178-19257
5 months ago
178-19258
5 months ago
6-21105
6 days
18748 FR-vdash-bot
author:FR-vdash-bot
refactor: deprecate `ContinuousLinearMapClass` --- - [ ] depends on: #18689 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-topology merge-conflict
label:t-algebra$
115/49 Mathlib/Analysis/CStarAlgebra/Spectrum.lean,Mathlib/Analysis/LocallyConvex/WeakOperatorTopology.lean,Mathlib/Analysis/Normed/Algebra/Spectrum.lean,Mathlib/Analysis/Normed/Operator/LinearIsometry.lean,Mathlib/Topology/Algebra/Module/Basic.lean,Mathlib/Topology/Algebra/Module/CharacterSpace.lean,Mathlib/Topology/Algebra/Module/FiniteDimension.lean,Mathlib/Topology/Algebra/Module/StrongTopology.lean,Mathlib/Topology/Algebra/Module/WeakDual.lean,Mathlib/Topology/Homeomorph.lean 10 5 ['FR-vdash-bot', 'github-actions', 'leanprover-bot', 'mathlib4-dependent-issues-bot'] nobody
175-21786
5 months ago
175-21789
5 months ago
0-989
16 minutes
20527 trivial1711
author:trivial1711
refactor(Topology/UniformSpace/Completion): more descriptive names for `α → Completion α` - We rename the various maps `α → Completion α` in order to make their names more consistent. - Let `α` be a uniform space. We rename the uniformly continuous function `α → Completion α` from `UniformSpace.Completion.coe'` to `UniformSpace.Completion.coe`. - Let `α` be a uniform additive group. We rename the additive group homomorphism `α →+ Completion α` from `UniformSpace.Completion.toCompl` to `UniformSpace.Completion.coeAddHom`. - Let `α` be a uniform ring. The ring homomorphism `α →+* Completion α` is called `UniformSpace.Completion.coeRingHom`; its name is unchanged. - Let `α` be a normed space over a field `𝕜`. We rename the linear isometry `α →ₗᵢ[𝕜] Completion α` from `UniformSpace.Completion.toComplₗᵢ` to `UniformSpace.Completion.coeₗᵢ`. - Let `α` be a normed space over a field `𝕜`. We rename the continuous linear map `α →L[𝕜] Completion α` from `UniformSpace.Completion.toComplL` to `UniformSpace.Completion.coeL`. - Let `α` be a normed additive group. We rename the norm preserving homomorphism `NormedAddGroupHom α (Completion α)` from `NormedAddCommGroup.toCompl` to `UniformSpace.Completion.coeNormedAddGroupHom`. - We analogously rename some other theorems. - We add some trivial theorems (all of which are proved by `rfl`) that state that the functions considered above are equal. We give all of them the `simp` and `norm_cast` attributes. - We add a new theorem `UniformSpace.Completion.coeAddHom_eq_coe` that states that `UniformSpace.Completion.coeAddHom` and `UniformSpace.Completion.coe` are equal as functions. - We similarly add a new theorem `UniformSpace.Completion.coeRingHom_eq_coe`. - We rename the theorem `UniformSpace.Completion.coe_toComplₗᵢ` to `UniformSpace.Completion.coeₗᵢ_eq_coe`. - We rename the theorem `UniformSpace.Completion.coe_toComplL` to `UniformSpace.Completion.coeL_eq_coe`. - We similarly add a new theorem `UniformSpace.Completion.coeNormedAddGroupHom_eq_coe`. - We change all occurrences of the string `((↑) : α → Completion α)` to `(coe : α → Completion α)` or just `coe`. - We put the statements of some theorems into simp normal form by using the plain function `coe` rather than the homomorphisms that carry more structure. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology merge-conflict 130/92 Mathlib/Analysis/Analytic/Uniqueness.lean,Mathlib/Analysis/Calculus/FDeriv/Analytic.lean,Mathlib/Analysis/Complex/AbsMax.lean,Mathlib/Analysis/Complex/Liouville.lean,Mathlib/Analysis/InnerProductSpace/Completion.lean,Mathlib/Analysis/Normed/Group/HomCompletion.lean,Mathlib/Analysis/Normed/Module/Completion.lean,Mathlib/Analysis/SpecialFunctions/NonIntegrable.lean,Mathlib/MeasureTheory/Integral/IntegralEqImproper.lean,Mathlib/Topology/Algebra/GroupCompletion.lean,Mathlib/Topology/Algebra/InfiniteSum/GroupCompletion.lean,Mathlib/Topology/Algebra/InfiniteSum/Nonarchimedean.lean,Mathlib/Topology/Algebra/Nonarchimedean/Completion.lean,Mathlib/Topology/Algebra/UniformRing.lean,Mathlib/Topology/Category/UniformSpace.lean,Mathlib/Topology/MetricSpace/Completion.lean,Mathlib/Topology/UniformSpace/Completion.lean 17 4 ['eric-wieser', 'github-actions', 'trivial1711'] nobody
147-18579
4 months ago
147-18579
4 months ago
6-66637
6 days
18474 FR-vdash-bot
author:FR-vdash-bot
perf: lower the priority of `*WithOne.to*` instances --- From #7873. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data slow-typeclass-synthesis t-algebra merge-conflict
label:t-algebra$
9/2 Mathlib/Algebra/Polynomial/BigOperators.lean,Mathlib/Data/Int/Cast/Defs.lean,Mathlib/Data/Nat/Cast/Defs.lean 3 7 ['FR-vdash-bot', 'eric-wieser', 'github-actions', 'leanprover-bot'] nobody
145-5609
4 months ago
145-5609
4 months ago
76-67978
76 days
19091 Vierkantor
author:Vierkantor
chore(Algebra/MonoidAlgebra): split Defs.lean further This PR further splits the big file `MonoidAlgebra/Defs.lean` to focus on the ring structure on (`Add`)`MonoidAlgebra`. The following files have been split off: * `MonoidAlgebra/Lift.lean`: definition of `liftNC` * `MonoidAlgebra/MapDomain.lean`: definition of `mapDomain` * `MonoidAlgebra/Module.lean`: module structure (and some submodule results) * `MonoidAlgebra/Opposite.lean`: results on the `MulOpposite` ring structure I also changed one proof about scalar multiplication by natural numbers, so that it wouldn't need a full on module structure on `Finsupp`. This required adding a pair of lemmas on the definition of multiplying `Finsupp`s by natural numbers. --- - [ ] depends on: #19087 - [ ] depends on: #19205 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict
label:t-algebra$
883/560 Mathlib.lean,Mathlib/Algebra/MonoidAlgebra/Basic.lean,Mathlib/Algebra/MonoidAlgebra/Defs.lean,Mathlib/Algebra/MonoidAlgebra/Division.lean,Mathlib/Algebra/MonoidAlgebra/Lift.lean,Mathlib/Algebra/MonoidAlgebra/MapDomain.lean,Mathlib/Algebra/MonoidAlgebra/Module.lean,Mathlib/Algebra/MonoidAlgebra/Opposite.lean,Mathlib/Algebra/MonoidAlgebra/Support.lean,Mathlib/Algebra/Polynomial/Basic.lean,Mathlib/Data/Finsupp/Defs.lean,Mathlib/RingTheory/Polynomial/Opposites.lean 12 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
144-27126
4 months ago
144-27126
4 months ago
2-72196
2 days
20372 jvlmdr
author:jvlmdr
feat(MeasureTheory/Function): Add ContinuousLinearMap.bilinearCompLp(L) Introduce ContinuousLinearMap.bilinearCompLp and bilinearCompLpL. Generalize eLpNorm_le_eLpNorm_mul_eLpNorm theorems to include constant C in bound condition. --- Expect this may be useful for defining tempered distributions from functions in `L^p`. The definitions more or less follow `ContinuousLinearMap.compLp...`. Names are loosely analogous to `ContinuousLinearMap.bilinearComp` and `SchwartzMap.bilinLeftCLM`. Note: I preferred the spelling `hpqr : p⁻¹ + q⁻¹ = r⁻¹` with `f` in `L^p` and `g` in `L^q` to `hpqr : 1 / p = 1 / q + 1 / r`. It's easier to obtain from `ENNReal.IsConjExponent` too. A few questions: - [ ] I defined `bilinear{Left,Right}LpL` in addition to `bilinearCompLpL` because `LinearMap.mkContinuous₂` is marked as `noncomputable` and `LinearMap.mkContinuous` is not. Is this worth the extra definitions? (Note: This is not visible in the source due to `noncomputable section`.) - [ ] Should I use `C : ℝ` instead of `C : NNReal` for `eLpNorm_le_eLpNorm_mul_eLpNorm'_of_norm'`? - [ ] Is it going to be painful to have `[Fact (1 ≤ p)] [Fact (1 ≤ q)] [Fact (1 ≤ r)]`? I don't think there's a way to avoid it though. Maybe providing specialized versions for `p.IsConjExponent q` with `L^1`? Naming: - [ ] Is it satisfactory to add a `'` to the `eLpNorm_le_eLpNorm_mul_eLpNorm ` definitions in `CompareExp.lean` where `≤ ‖f x‖ * ‖g x‖` has been replaced with `≤ C * ‖f x‖ * ‖g x‖`? These could replace the existing theorems, although I don't want to break backwards compatibility. There are 5 instances: `eLpNorm_le_eLpNorm_top_mul_eLpNorm'`, `eLpNorm_le_eLpNorm_mul_eLpNorm_top'`, `eLpNorm'_le_eLpNorm'_mul_eLpNorm''`, `eLpNorm_le_eLpNorm_mul_eLpNorm_of_nnnorm'`, `eLpNorm_le_eLpNorm_mul_eLpNorm'_of_norm'` (I'm not sure why the existing theorem `eLpNorm_le_eLpNorm_mul_eLpNorm'_of_norm` has an internal `'`) - [ ] Is `bilinearLeftLpL` a suitable name? Other options: `bilinearCompLpLeftL`, `bilinearCompLeftLpL`, `bilinLeftLpL` (analogous to `SchwartzMap.bilinLeftCLM`) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-measure-probability merge-conflict 203/40 Mathlib/MeasureTheory/Function/LpSeminorm/CompareExp.lean,Mathlib/MeasureTheory/Function/LpSpace.lean 2 1 ['github-actions'] nobody
132-29866
4 months ago
132-29866
4 months ago
27-43617
27 days
21948 ChrisHughes24
author:ChrisHughes24
feat(ModelTheory): Formula.iSup and iInf --- This was a slightly controversial addition discussed in #20175 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-logic merge-conflict 24/7 Mathlib/ModelTheory/Semantics.lean,Mathlib/ModelTheory/Syntax.lean 2 5 ['YaelDillies', 'github-actions'] nobody
112-19326
3 months ago
112-19326
3 months ago
1-18127
1 day
18463 vihdzp
author:vihdzp
feat(SetTheory/Ordinal/Notation/FundamentalSequence): define type of fundamental sequences We define `Sequence α` as the type of sequences with length 0, 1, or `ω`, and give a basic API. A subsequent PR will introduce the notion of a (countable and computable) fundamental sequence and establish basic results. The goal of this is to generalize [`ONote.fundamentalSequence`](https://leanprover-community.github.io/mathlib4_docs/Mathlib/SetTheory/Ordinal/Notation.html#ONote.fundamentalSequence) to allow the construction of fundamental sequences for other ordinal notations. --- See [my ordinal notation repository](https://github.com/vihdzp/ordinal-notation/blob/a6fdd7fe7cb521e686ea271902e7e5496f1804d3/OrdinalNotation/Cantor.lean#L1218) for a demonstration of how this API looks in practice. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-set-theory t-order merge-conflict 174/1 Mathlib.lean,Mathlib/SetTheory/Ordinal/Notation/Cantor.lean,Mathlib/SetTheory/Ordinal/Notation/FundamentalSequence.lean 3 19 ['YnirPaz', 'b-mehta', 'github-actions', 'vihdzp'] nobody
110-54008
3 months ago
110-54008
3 months ago
52-25108
52 days
21099 chrisflav
author:chrisflav
chore(RingTheory/Generators): use unification hints for variables and relations When working with generators and presentations, we rely on the `MvPolynomial` API, but since the type of variables is bundled in `Generators R S`, many lemmas don't apply with `rw` or `simp`, because they can't see through the definition of `vars` in constructions such as `Generators.comp` and `Generators.localizationAway`. A possible approach is to make all of these constructions `abbrev`s, but this causes `simp` to also unfold `val` which is not always desirable. More generally, it is then harder to predict how instance search and `simp` behave. This approach is tried in #21050, but causes many regressions. This approach is less invasive, as it uses `unif_hint` to unify the `vars` (and `rels`) fields of constructions with the correct type. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict
label:t-algebra$
231/91 Mathlib/Algebra/Module/Presentation/Differentials.lean,Mathlib/RingTheory/Generators.lean,Mathlib/RingTheory/Kaehler/JacobiZariski.lean,Mathlib/RingTheory/Presentation.lean,Mathlib/RingTheory/Smooth/StandardSmooth.lean 5 16 ['chrisflav', 'erdOne', 'github-actions', 'leanprover-bot', 'mattrobball'] nobody
106-12844
3 months ago
106-12844
3 months ago
27-75210
27 days
13964 pechersky
author:pechersky
feat(Data/DigitExpansion): begin defining variant of reals without rationals Based on a de Bruijn 1976 paper. This file is just the basic definition of a digit expansion. Will be followed up with furhter constructions. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data merge-conflict 518/0 Mathlib.lean,Mathlib/Data/DigitExpansion/Defs.lean,docs/references.bib 3 11 ['eric-wieser', 'github-actions', 'kim-em', 'pechersky'] dupuisf
assignee:dupuisf
98-15949
3 months ago
225-32457
7 months ago
129-57991
129 days
21339 vihdzp
author:vihdzp
fix(Data/List/Lex): remove duplicate `List.LE` instance Mathlib currently duplicates the Lean core instance for `≤` in lists in an incompatible way. We delete this duplicate instance. See [Zulip](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Two.20.60List.2ELE.60.20instances.3F/near/497241115). --- This is a very quick and dirty fix. Core Lean provides all of the theorems we need to prove `≤` forms a linear order, but it provides them in terms of `Std` relation typeclasses which currently see no use in Mathlib. I've added the instances that were required to get the list theorems working. In the future, we really ought to unify the core and Mathlib relation typeclasses. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data merge-conflict 24/22 Mathlib/Data/List/Lex.lean,Mathlib/Data/String/Basic.lean,Mathlib/Topology/Category/Profinite/Nobeling.lean 3 1 ['github-actions'] nobody
98-11736
3 months ago
98-11736
3 months ago
16-65973
16 days
21959 BGuillemet
author:BGuillemet
feat(Topology/ContinuousMap): Stone-Weierstrass theorem for MvPolynomial Add the subalgebra of multivariate polynomials and prove it separates points, on the same model as `ContinuousMap/Polynomial.lean`. Prove the Stone-Weierstrass theorem and some variations for multivariate polynomials. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-topology merge-conflict 285/1 Mathlib.lean,Mathlib/Topology/ContinuousMap/MvPolynomial.lean,Mathlib/Topology/ContinuousMap/StoneWeierstrass.lean 3 1 ['github-actions'] nobody
96-15887
3 months ago
96-15887
3 months ago
16-76141
16 days
22660 Ruben-VandeVelde
author:Ruben-VandeVelde
chore: follow naming convention around Group.IsNilpotent --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict
label:t-algebra$
133/67 Mathlib/GroupTheory/Frattini.lean,Mathlib/GroupTheory/Nilpotent.lean,Mathlib/GroupTheory/SpecificGroups/ZGroup.lean 3 1 ['github-actions'] nobody
84-38142
2 months ago
84-38142
2 months ago
10-48025
10 days
21856 vihdzp
author:vihdzp
chore(SetTheory/Cardinal/Basic): generalize universes of `sum_le_iSup_lift` We prove a more general version of the lemma which talks about families `ι → Cardinal.{v}` with `Small.{v} ι`, rather than just families `f : ι → Cardinal.{max u v}` with `ι : Type v`. We keep the old version, as it's seemingly more useful under common circumstances. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-set-theory merge-conflict 16/10 Mathlib/SetTheory/Cardinal/Basic.lean 1 6 ['b-mehta', 'github-actions', 'vihdzp'] nobody
83-29376
2 months ago
83-29376
2 months ago
32-26420
32 days
22027 vihdzp
author:vihdzp
chore(SetTheory/Ordinal/FixedPoint); review `Ordinal.nfp` API This PR does the following: - add `iff` variants of various theorems, renaming some in the process - weaken some assumptions slightly - golf throughout --- - [x] depends on: #22017 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-set-theory merge-conflict 64/61 Mathlib/Logic/Equiv/List.lean,Mathlib/SetTheory/Ordinal/FixedPoint.lean 2 3 ['github-actions', 'grunweg', 'mathlib4-dependent-issues-bot'] nobody
64-82294
2 months ago
67-49254
2 months ago
43-68322
43 days
13861 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`. 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 do some light refactoring for succinctness, and put this any related preexisting lemmas in a new file to not trigger the linter. Needed by #12664 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data merge-conflict 204/62 Mathlib.lean,Mathlib/Algebra/Category/MonCat/Adjunctions.lean,Mathlib/Data/Finsupp/Basic.lean,Mathlib/Data/Finsupp/Option.lean,Mathlib/Data/Finsupp/Single.lean,Mathlib/LinearAlgebra/Finsupp/LinearCombination.lean 6 1 ['github-actions'] nobody
63-80879
2 months ago
63-80879
2 months ago
12-6613
12 days
21858 vihdzp
author:vihdzp
refactor(SetTheory/Ordinal/FixedPoint): redefine `Ordinal.deriv` We previously defined the [ordinal derivative](https://en.wikipedia.org/wiki/Normal_function#Properties) of a function as the unique normal function satisfying `deriv f 0 = nfp f 0` and `deriv f (o + 1) = nfp f (deriv f o)` (where `nfp f a` is the next fixed point of `f` that's `≥ a`). The motivation here was to give a "nice" junk value on non-normal functions (the function is normal no matter what). However, in practice, this definition makes it unwieldy to prove things, by either requiring a tedious zero/successor/limit argument, or requiring one to rewrite `deriv f = enumOrd (fixedPoints f)`. We can instead define `deriv f = enumOrd (fixedPoints f)`. At the cost of giving "worse" junk values (which we have no legitimate uses of), we're able to much more easily prove all the expected properties in the standard case where `f` is a normal function. Finally, we do some drive-by API cleanup. --- - [ ] depends on: #21860 - [ ] depends on: #21970 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-set-theory merge-conflict 216/262 Mathlib/Logic/Equiv/List.lean,Mathlib/SetTheory/Cardinal/Cofinality.lean,Mathlib/SetTheory/Ordinal/Enum.lean,Mathlib/SetTheory/Ordinal/FixedPoint.lean,Mathlib/SetTheory/Ordinal/Principal.lean,Mathlib/SetTheory/Ordinal/Veblen.lean 6 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
63-80341
2 months ago
63-80343
2 months ago
0-1601
26 minutes
22701 ctchou
author:ctchou
feat(Combinatorics): the Katona circle method This file formalizes the Katona circle method. From PlainCombi (LeanCamCombi): https://github.com/YaelDillies/LeanCamCombi/blob/master/LeanCamCombi/PlainCombi/KatonaCircle.lean Co-authored-by: Yaël Dillies new-contributor t-combinatorics merge-conflict 121/0 Mathlib.lean,Mathlib/Combinatorics/KatonaCircle.lean 2 1 ['github-actions'] nobody
63-78056
2 months ago
63-78056
2 months ago
30-8337
30 days
23411 PatrickMassot
author:PatrickMassot
chore: remove finiteness from Order.Filter.Lift Co-authored-by: Anatole Dedecker --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) longest-pole t-topology merge-conflict 48/21 Mathlib/Dynamics/TopologicalEntropy/DynamicalEntourage.lean,Mathlib/Order/Filter/Basic.lean,Mathlib/Order/Filter/Finite.lean,Mathlib/Order/Filter/Lift.lean,Mathlib/Order/Filter/SmallSets.lean,Mathlib/Topology/Algebra/ContinuousMonoidHom.lean,Mathlib/Topology/Basic.lean 7 4 ['Vierkantor', 'github-actions', 'kim-em', 'leanprover-community-bot-assistant'] nobody
62-38370
2 months ago
62-57939
2 months ago
10-21608
10 days
21488 imbrem
author:imbrem
feat(CategoryTheory/Monoidal): premonoidal categories Add support for premonoidal categories --- Still want to add support for: - Premonoidal braided/symmetric categories - The monoidal coherence theorem, which I've already ported in my `discretion` library - The `coherence` tactic, which should work fine for premonoidal categories too but wanted to get this in front of reviewers ASAP to make sure my general approach was alright [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-category-theory merge-conflict 900/361 Mathlib/Algebra/Category/ModuleCat/Presheaf/Monoidal.lean,Mathlib/CategoryTheory/Bicategory/End.lean,Mathlib/CategoryTheory/GradedObject/Monoidal.lean,Mathlib/CategoryTheory/Localization/Monoidal.lean,Mathlib/CategoryTheory/Monoidal/Braided/Basic.lean,Mathlib/CategoryTheory/Monoidal/Category.lean,Mathlib/CategoryTheory/Monoidal/Center.lean,Mathlib/CategoryTheory/Monoidal/CoherenceLemmas.lean,Mathlib/CategoryTheory/Monoidal/Discrete.lean,Mathlib/CategoryTheory/Monoidal/End.lean,Mathlib/CategoryTheory/Monoidal/Free/Basic.lean,Mathlib/CategoryTheory/Monoidal/Functor.lean,Mathlib/CategoryTheory/Monoidal/FunctorCategory.lean,Mathlib/CategoryTheory/Monoidal/Mon_.lean,Mathlib/CategoryTheory/Monoidal/Opposite.lean,Mathlib/CategoryTheory/Monoidal/Transport.lean,Mathlib/Tactic/CategoryTheory/Monoidal/Datatypes.lean,Mathlib/Tactic/CategoryTheory/Monoidal/Normalize.lean,Mathlib/Tactic/CategoryTheory/Monoidal/PureCoherence.lean,Mathlib/Tactic/CategoryTheory/MonoidalComp.lean,MathlibTest/StringDiagram.lean 21 9 ['YaelDillies', 'github-actions', 'grunweg', 'imbrem', 'kim-em', 'leanprover-community-bot-assistant'] nobody
61-24289
2 months ago
61-24290
2 months ago
58-20339
58 days
21525 sinhp
author:sinhp
feat(CategoryTheory): Locally Cartesian Closed Categories (Prelim) This PR defines the basic preliminaries for defining locally cartesian closed categories (LCCCs). In particular, using the calculus of mates we define certain natural isomorphisms involving `Over.star` and `Over.pullback` which will be crucial in defining the right adjoint to the pullback functor in the development of LCCCs. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-category-theory merge-conflict 338/24 Mathlib/CategoryTheory/Comma/Over/Basic.lean,Mathlib/CategoryTheory/Comma/Over/Pullback.lean,Mathlib/CategoryTheory/Galois/Examples.lean 3 13 ['b-mehta', 'github-actions', 'joelriou', 'leanprover-community-bot-assistant', 'sinhp'] nobody
61-24287
2 months ago
61-24289
2 months ago
43-83249
43 days
16314 FR-vdash-bot
author:FR-vdash-bot
chore(Data/Quot): deprecate `ind*'` APIs --- - [x] depends on: #16264 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data merge-conflict 247/287 Counterexamples/CliffordAlgebraNotInjective.lean,Mathlib/Algebra/Colimit/Module.lean,Mathlib/Algebra/Lie/Quotient.lean,Mathlib/Algebra/Module/Torsion.lean,Mathlib/Algebra/RingQuot.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Angle.lean,Mathlib/CategoryTheory/ConnectedComponents.lean,Mathlib/CategoryTheory/Subobject/Basic.lean,Mathlib/CategoryTheory/Subobject/FactorThru.lean,Mathlib/CategoryTheory/Subobject/Lattice.lean,Mathlib/Computability/Reduce.lean,Mathlib/Computability/Tape.lean,Mathlib/Data/List/Cycle.lean,Mathlib/Data/Multiset/MapFold.lean,Mathlib/Data/Multiset/ZeroCons.lean,Mathlib/Data/Quot.lean,Mathlib/Data/Setoid/Basic.lean,Mathlib/Data/Setoid/Partition.lean,Mathlib/FieldTheory/Fixed.lean,Mathlib/GroupTheory/Complement.lean,Mathlib/GroupTheory/Congruence/Basic.lean,Mathlib/GroupTheory/Congruence/Defs.lean,Mathlib/GroupTheory/Congruence/Hom.lean,Mathlib/GroupTheory/Coset/Basic.lean,Mathlib/GroupTheory/Coset/Defs.lean,Mathlib/GroupTheory/FreeAbelianGroup.lean,Mathlib/GroupTheory/GroupAction/Basic.lean,Mathlib/GroupTheory/GroupAction/Defs.lean,Mathlib/GroupTheory/GroupAction/Quotient.lean,Mathlib/GroupTheory/Index.lean,Mathlib/GroupTheory/MonoidLocalization/Basic.lean,Mathlib/GroupTheory/PGroup.lean,Mathlib/GroupTheory/Perm/Cycle/Concrete.lean,Mathlib/GroupTheory/PresentedGroup.lean,Mathlib/GroupTheory/QuotientGroup/Basic.lean,Mathlib/GroupTheory/QuotientGroup/Defs.lean,Mathlib/GroupTheory/SchurZassenhaus.lean,Mathlib/GroupTheory/Sylow.lean,Mathlib/LinearAlgebra/Alternating/DomCoprod.lean,Mathlib/LinearAlgebra/Projectivization/Basic.lean,Mathlib/LinearAlgebra/Quotient/Basic.lean,Mathlib/LinearAlgebra/Quotient/Defs.lean,Mathlib/MeasureTheory/Function/AEEqFun.lean,Mathlib/NumberTheory/Padics/PadicNumbers.lean,Mathlib/NumberTheory/RamificationInertia/Basic.lean,Mathlib/Order/Antisymmetrization.lean,Mathlib/Order/Category/PartOrd.lean,Mathlib/Order/Filter/Germ/Basic.lean,Mathlib/RepresentationTheory/GroupCohomology/Hilbert90.lean,Mathlib/RingTheory/AdicCompletion/Algebra.lean,Mathlib/RingTheory/AdicCompletion/Basic.lean,Mathlib/RingTheory/AdicCompletion/Functoriality.lean,Mathlib/RingTheory/AdjoinRoot.lean,Mathlib/RingTheory/Congruence/Basic.lean,Mathlib/RingTheory/Flat/FaithfullyFlat/Basic.lean,Mathlib/RingTheory/GradedAlgebra/HomogeneousLocalization.lean,Mathlib/RingTheory/Ideal/Cotangent.lean,Mathlib/RingTheory/Ideal/Norm/AbsNorm.lean,Mathlib/RingTheory/Ideal/Quotient/Basic.lean,Mathlib/RingTheory/Ideal/Quotient/Defs.lean,Mathlib/RingTheory/Ideal/Quotient/Operations.lean,Mathlib/RingTheory/Valuation/Quotient.lean,Mathlib/Topology/Algebra/Group/TopologicalAbelianization.lean,Mathlib/Topology/Algebra/InfiniteSum/Module.lean,Mathlib/Topology/Separation/Basic.lean 65 4 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
55-49253
1 month ago
55-49255
1 month ago
55-52030
55 days
23211 Parcly-Taxel
author:Parcly-Taxel
chore: automatically deprime common `induction'` uses Replace `induction'` with `induction` for the following targets: ```python rep_dict = {("Nat", "~", 2): [("zero", 0), ("succ", 2)], ("Nat", "strong_induction_on", 1): [("h", 2)], ("Nat", "case_strong_induction_on", 2): [("hz", 0), ("hi", 2)], ("Nat", "le_induction", 2): [("base", 0), ("succ", 3)], ("List", "~", 2): [("nil", 0), ("cons", 3)], ("List", "reverseRecOn", 2): [("nil", 0), ("append_singleton", 3)], ("Multiset", "induction_on", 2): [("empty", 0), ("cons", 3)], ("Finset", "induction", 2): [("empty", 0), ("@insert", 4)], ("Finset", "induction_on", 2): [("empty", 0), ("@insert", 4)], ("MvPolynomial", "induction_on'", 2): [("monomial", 2), ("add", 4)], ("MvPolynomial", "induction_on", 3): [("C", 1), ("add", 4), ("mul_X", 3)]} ``` The script and the data file used can be found [here](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/The.20plan.20to.20remove.20induction'/near/508218834). tech debt merge-conflict 2189/1565 Archive/Imo/Imo1977Q6.lean,Archive/Imo/Imo2006Q5.lean,Archive/Imo/Imo2013Q1.lean,Archive/Imo/Imo2013Q5.lean,Archive/Imo/Imo2019Q4.lean,Archive/Imo/Imo2024Q1.lean,Archive/MiuLanguage/DecisionSuf.lean,Archive/Sensitivity.lean,Archive/Wiedijk100Theorems/FriendshipGraphs.lean,Archive/Wiedijk100Theorems/Partition.lean,Mathlib/Algebra/Algebra/Subalgebra/Lattice.lean,Mathlib/Algebra/BigOperators/Group/List/Lemmas.lean,Mathlib/Algebra/Group/Conj.lean,Mathlib/Algebra/Group/ForwardDiff.lean,Mathlib/Algebra/Group/Pointwise/Finset/Basic.lean,Mathlib/Algebra/Group/Pointwise/Set/BigOperators.lean,Mathlib/Algebra/Group/Pointwise/Set/Finite.lean,Mathlib/Algebra/Group/Pointwise/Set/ListOfFn.lean,Mathlib/Algebra/Lie/Solvable.lean,Mathlib/Algebra/Module/PID.lean,Mathlib/Algebra/Order/BigOperators/Group/List.lean,Mathlib/Algebra/Order/CauSeq/BigOperators.lean,Mathlib/Algebra/Order/Group/Multiset.lean,Mathlib/Algebra/Polynomial/BigOperators.lean,Mathlib/Algebra/Polynomial/Degree/Lemmas.lean,Mathlib/Algebra/Polynomial/Derivative.lean,Mathlib/Algebra/Polynomial/EraseLead.lean,Mathlib/Algebra/Polynomial/Eval/Defs.lean,Mathlib/Algebra/Polynomial/HasseDeriv.lean,Mathlib/Algebra/Ring/Subring/Basic.lean,Mathlib/Algebra/Tropical/BigOperators.lean,Mathlib/AlgebraicTopology/DoldKan/Decomposition.lean,Mathlib/AlgebraicTopology/DoldKan/Degeneracies.lean,Mathlib/AlgebraicTopology/DoldKan/Projections.lean,Mathlib/Analysis/Analytic/Composition.lean,Mathlib/Analysis/Analytic/Constructions.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/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/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/Log/Base.lean,Mathlib/Analysis/SpecialFunctions/Pow/Deriv.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/EulerSineProd.lean,Mathlib/CategoryTheory/ComposableArrows.lean,Mathlib/CategoryTheory/Extensive.lean,Mathlib/CategoryTheory/Filtered/Basic.lean,Mathlib/CategoryTheory/Limits/VanKampen.lean,Mathlib/CategoryTheory/Triangulated/TStructure/Basic.lean,Mathlib/Computability/Ackermann.lean,Mathlib/Computability/DFA.lean,Mathlib/Computability/EpsilonNFA.lean,Mathlib/Computability/Language.lean,Mathlib/Computability/NFA.lean,Mathlib/Computability/Partrec.lean,Mathlib/Computability/PartrecCode.lean,Mathlib/Computability/PostTuringMachine.lean,Mathlib/Computability/Primrec.lean,Mathlib/Computability/RegularExpressions.lean,Mathlib/Computability/TMConfig.lean,Mathlib/Computability/TMToPartrec.lean,Mathlib/Computability/Tape.lean,Mathlib/Control/LawfulFix.lean,Mathlib/Data/Complex/Exponential.lean,Mathlib/Data/Countable/Basic.lean,Mathlib/Data/DFinsupp/Defs.lean,Mathlib/Data/DFinsupp/WellFounded.lean,Mathlib/Data/Fin/Tuple/Basic.lean,Mathlib/Data/Fin/Tuple/NatAntidiagonal.lean,Mathlib/Data/Finmap.lean,Mathlib/Data/Finset/Fold.lean,Mathlib/Data/Finset/Image.lean,Mathlib/Data/Finset/Lattice/Fold.lean,Mathlib/Data/Finset/Lattice/Lemmas.lean,Mathlib/Data/Finset/Lattice/Pi.lean,Mathlib/Data/Finset/Max.lean,Mathlib/Data/Finset/NAry.lean,Mathlib/Data/Finset/NoncommProd.lean,Mathlib/Data/Finset/Sym.lean,Mathlib/Data/Finsupp/BigOperators.lean,Mathlib/Data/Fintype/Basic.lean,Mathlib/Data/Fintype/Card.lean,Mathlib/Data/Fintype/EquivFin.lean,Mathlib/Data/Fintype/Fin.lean 283 2 ['github-actions', 'leanprover-community-bot-assistant'] nobody
55-47427
1 month ago
55-47429
1 month ago
10-65025
10 days
13795 FR-vdash-bot
author:FR-vdash-bot
perf(Algebra/{Group, GroupWithZero, Ring}/InjSurj): reduce everything --- - [ ] depends on: #15192 - [ ] depends on: #15476 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict
label:t-algebra$
340/194 Mathlib/Algebra/Equiv/TransferInstance.lean,Mathlib/Algebra/Group/InjSurj.lean,Mathlib/Algebra/GroupWithZero/Action/Defs.lean,Mathlib/Algebra/GroupWithZero/Action/End.lean,Mathlib/Algebra/GroupWithZero/InjSurj.lean,Mathlib/Algebra/Module/Defs.lean,Mathlib/Algebra/Module/RingHom.lean,Mathlib/Algebra/Ring/InjSurj.lean,scripts/noshake.json 9 35 ['FR-vdash-bot', 'MichaelStollBayreuth', 'eric-wieser', 'github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mattrobball'] nobody
55-41568
1 month ago
55-41570
1 month ago
52-31623
52 days
15483 FR-vdash-bot
author:FR-vdash-bot
chore(GroupTheory/Coset): reduce defeq abuse --- - [x] depends on: #15482 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict
label:t-algebra$
114/60 Mathlib/GroupTheory/Commensurable.lean,Mathlib/GroupTheory/Coset.lean,Mathlib/GroupTheory/QuotientGroup.lean,Mathlib/LinearAlgebra/Alternating/DomCoprod.lean,Mathlib/MeasureTheory/Measure/Haar/Quotient.lean,Mathlib/Topology/Algebra/Group/Compact.lean 6 14 ['FR-vdash-bot', 'eric-wieser', 'github-actions', 'grunweg', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'mattrobball', 'mergify', 'urkud'] nobody
54-80546
1 month ago
303-32476
9 months ago
4-79214
4 days
20567 grunweg
author:grunweg
feat(Cache): two small features - add an informational message to the get command (when run without arguments): when more than 80% of all cache files present were not used in the last command, tell the user about the `clean` command --- - [ ] depends on #20568 (for the first feature) - [ ] TODO: re-design this feature and the clean command: if there are N local copies of mathlib, cache should have a pointer to all of them - to avoid clearing all N-1 from inside the last local copy [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta merge-conflict 38/2 Cache/Main.lean 1 11 ['Julian', 'arthurpaulino', 'fpvandoorn', 'github-actions', 'grunweg'] nobody
52-84649
1 month ago
52-84649
1 month ago
1-17369
1 day
23859 urkud
author:urkud
feat(Topology/../Order/Field): generalize to `Semifield` .. from a linear ordered field to a linear ordered semifield--- - [ ] depends on: #23857 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology merge-conflict 245/219 Mathlib/Algebra/Order/Group/Pointwise/Interval.lean,Mathlib/Analysis/BoxIntegral/Box/SubboxInduction.lean,Mathlib/Topology/Algebra/Order/Field.lean,Mathlib/Topology/Order/Basic.lean 4 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
48-37163
1 month ago
48-37166
1 month ago
0-265
4 minutes
23810 b-reinke
author:b-reinke
chore(Order/Interval): generalize succ/pred lemmas to partial orders Many lemmas in `Mathlib/Order/Interval/Set/SuccPred.lean`and `Mathlib/Order/Interval/Finset/SuccPred.lean` also work for partial orders. They are generalized in this PR by introducing different sections for `PartialOrder` and `LinearOrder` assumptions in the respective files. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order merge-conflict 231/89 Mathlib/Order/Interval/Finset/SuccPred.lean,Mathlib/Order/Interval/Set/SuccPred.lean 2 2 ['github-actions', 'leanprover-community-bot-assistant'] nobody
46-13938
1 month ago
46-13940
1 month ago
16-29623
16 days
24285 madvorak
author:madvorak
chore(Algebra/*-{Category,Homology}): remove unnecessary universe variables Discussions: https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Call.20for.20help.3A.20technical.2F.20organisational.20debt/with/513620128 https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Algebra.20and.20.60Type*.60/with/513558902 https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Task.2026.3A.20Replace.20Type.20u.20by.20Type*.20wherever.20possible/with/513592993 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict
label:t-algebra$
542/916 Mathlib/Algebra/AddTorsor/Basic.lean,Mathlib/Algebra/Algebra/Defs.lean,Mathlib/Algebra/Algebra/Equiv.lean,Mathlib/Algebra/Algebra/Field.lean,Mathlib/Algebra/Algebra/Hom.lean,Mathlib/Algebra/Algebra/Operations.lean,Mathlib/Algebra/Algebra/Spectrum/Basic.lean,Mathlib/Algebra/Algebra/Subalgebra/Lattice.lean,Mathlib/Algebra/Algebra/Subalgebra/Tower.lean,Mathlib/Algebra/Algebra/Tower.lean,Mathlib/Algebra/Central/Basic.lean,Mathlib/Algebra/Central/Defs.lean,Mathlib/Algebra/Central/TensorProduct.lean,Mathlib/Algebra/CharP/Pi.lean,Mathlib/Algebra/CharP/Quotient.lean,Mathlib/Algebra/CharP/Subring.lean,Mathlib/Algebra/DirectSum/Algebra.lean,Mathlib/Algebra/DirectSum/Basic.lean,Mathlib/Algebra/DirectSum/Finsupp.lean,Mathlib/Algebra/DirectSum/Module.lean,Mathlib/Algebra/EuclideanDomain/Basic.lean,Mathlib/Algebra/EuclideanDomain/Defs.lean,Mathlib/Algebra/Field/Basic.lean,Mathlib/Algebra/Field/Defs.lean,Mathlib/Algebra/Field/IsField.lean,Mathlib/Algebra/Field/MinimalAxioms.lean,Mathlib/Algebra/Field/Subfield/Basic.lean,Mathlib/Algebra/Field/Subfield/Defs.lean,Mathlib/Algebra/FreeNonUnitalNonAssocAlgebra.lean,Mathlib/Algebra/Group/Conj.lean,Mathlib/Algebra/Group/Defs.lean,Mathlib/Algebra/Group/Equiv/Finite.lean,Mathlib/Algebra/Group/Ext.lean,Mathlib/Algebra/Group/Hom/End.lean,Mathlib/Algebra/Group/Hom/Instances.lean,Mathlib/Algebra/Group/Invertible/Basic.lean,Mathlib/Algebra/Group/Invertible/Defs.lean,Mathlib/Algebra/Group/Pi/Basic.lean,Mathlib/Algebra/Group/Pi/Lemmas.lean,Mathlib/Algebra/Group/TypeTags/Basic.lean,Mathlib/Algebra/Group/TypeTags/Finite.lean,Mathlib/Algebra/Group/TypeTags/Hom.lean,Mathlib/Algebra/Group/Units/Basic.lean,Mathlib/Algebra/Group/Units/Defs.lean,Mathlib/Algebra/Group/Units/Hom.lean,Mathlib/Algebra/Group/WithOne/Basic.lean,Mathlib/Algebra/Group/WithOne/Defs.lean,Mathlib/Algebra/GroupWithZero/Action/Pi.lean,Mathlib/Algebra/GroupWithZero/Defs.lean,Mathlib/Algebra/GroupWithZero/Invertible.lean,Mathlib/Algebra/GroupWithZero/NeZero.lean,Mathlib/Algebra/Lie/Abelian.lean,Mathlib/Algebra/Lie/Basic.lean,Mathlib/Algebra/Lie/CartanMatrix.lean,Mathlib/Algebra/Lie/CartanSubalgebra.lean,Mathlib/Algebra/Lie/Character.lean,Mathlib/Algebra/Lie/Classical.lean,Mathlib/Algebra/Lie/DirectSum.lean,Mathlib/Algebra/Lie/Free.lean,Mathlib/Algebra/Lie/Ideal.lean,Mathlib/Algebra/Lie/IdealOperations.lean,Mathlib/Algebra/Lie/Matrix.lean,Mathlib/Algebra/Lie/Nilpotent.lean,Mathlib/Algebra/Lie/NonUnitalNonAssocAlgebra.lean,Mathlib/Algebra/Lie/OfAssociative.lean,Mathlib/Algebra/Lie/Quotient.lean,Mathlib/Algebra/Lie/SkewAdjoint.lean,Mathlib/Algebra/Lie/Solvable.lean,Mathlib/Algebra/Lie/Subalgebra.lean,Mathlib/Algebra/Lie/Submodule.lean,Mathlib/Algebra/Lie/TensorProduct.lean,Mathlib/Algebra/Lie/UniversalEnveloping.lean,Mathlib/Algebra/Module/Basic.lean,Mathlib/Algebra/Module/CharacterModule.lean,Mathlib/Algebra/Module/DedekindDomain.lean,Mathlib/Algebra/Module/Defs.lean,Mathlib/Algebra/Module/End.lean,Mathlib/Algebra/Module/Equiv/Opposite.lean,Mathlib/Algebra/Module/Lattice.lean,Mathlib/Algebra/Module/LinearMap/Basic.lean,Mathlib/Algebra/Module/LinearMap/Defs.lean,Mathlib/Algebra/Module/LinearMap/End.lean,Mathlib/Algebra/Module/LocalizedModule/Basic.lean,Mathlib/Algebra/Module/MinimalAxioms.lean,Mathlib/Algebra/Module/NatInt.lean,Mathlib/Algebra/Module/Opposite.lean,Mathlib/Algebra/Module/Pi.lean,Mathlib/Algebra/Module/Presentation/Differentials.lean,Mathlib/Algebra/Module/Presentation/Tensor.lean,Mathlib/Algebra/Module/Rat.lean,Mathlib/Algebra/Module/RingHom.lean,Mathlib/Algebra/Module/Submodule/Basic.lean,Mathlib/Algebra/Module/Torsion.lean,Mathlib/Algebra/MonoidAlgebra/Basic.lean,Mathlib/Algebra/MonoidAlgebra/Defs.lean,Mathlib/Algebra/MonoidAlgebra/Support.lean,Mathlib/Algebra/MvPolynomial/Basic.lean,Mathlib/Algebra/MvPolynomial/CommRing.lean,Mathlib/Algebra/MvPolynomial/Degrees.lean,Mathlib/Algebra/MvPolynomial/Equiv.lean 182 22 ['erdOne', 'github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'madvorak', 'mattrobball'] nobody
46-2635
1 month ago
46-2636
1 month ago
2-12022
2 days
23621 FR-vdash-bot
author:FR-vdash-bot
chore: deprecate `LinearOrderedComm{Monoid, Group}WithZero` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) - [x] depends on: #20676 t-order t-algebra merge-conflict
label:t-algebra$
261/205 Archive/Imo/Imo1998Q2.lean,Counterexamples/LinearOrderWithPosMulPosEqZero.lean,Mathlib/Algebra/Order/Field/Canonical.lean,Mathlib/Algebra/Order/Field/Rat.lean,Mathlib/Algebra/Order/Floor/Ring.lean,Mathlib/Algebra/Order/GroupWithZero/Canonical.lean,Mathlib/Algebra/Order/GroupWithZero/Finset.lean,Mathlib/Algebra/Order/Hom/Monoid.lean,Mathlib/Algebra/Order/Nonneg/Field.lean,Mathlib/Algebra/Order/Nonneg/Ring.lean,Mathlib/Algebra/Order/Ring/Nat.lean,Mathlib/Combinatorics/Additive/PluenneckeRuzsa.lean,Mathlib/Combinatorics/SimpleGraph/Triangle/Basic.lean,Mathlib/Data/ENNReal/Basic.lean,Mathlib/Data/NNRat/Lemmas.lean,Mathlib/Data/NNReal/Defs.lean,Mathlib/Data/Rat/Cast/Order.lean,Mathlib/FieldTheory/IntermediateField/Adjoin/Defs.lean,Mathlib/FieldTheory/RatFunc/AsPolynomial.lean,Mathlib/GroupTheory/ArchimedeanDensely.lean,Mathlib/NumberTheory/EllipticDivisibilitySequence.lean,Mathlib/NumberTheory/FunctionField.lean,Mathlib/NumberTheory/Ostrowski.lean,Mathlib/RingTheory/Valuation/Archimedean.lean,Mathlib/RingTheory/Valuation/Basic.lean,Mathlib/RingTheory/Valuation/ExtendToLocalization.lean,Mathlib/RingTheory/Valuation/Integers.lean,Mathlib/RingTheory/Valuation/Integral.lean,Mathlib/RingTheory/Valuation/Minpoly.lean,Mathlib/RingTheory/Valuation/Quotient.lean,Mathlib/RingTheory/Valuation/RankOne.lean,Mathlib/RingTheory/Valuation/ValExtension.lean,Mathlib/RingTheory/Valuation/ValuationRing.lean,Mathlib/RingTheory/Valuation/ValuationSubring.lean,Mathlib/SetTheory/Cardinal/Order.lean,Mathlib/Topology/Algebra/Valued/LocallyCompact.lean,Mathlib/Topology/Algebra/Valued/NormedValued.lean,Mathlib/Topology/Algebra/Valued/ValuationTopology.lean,Mathlib/Topology/Algebra/Valued/ValuedField.lean,Mathlib/Topology/Algebra/Valued/WithVal.lean,Mathlib/Topology/Algebra/WithZeroTopology.lean,Mathlib/Topology/UnitInterval.lean,MathlibTest/instance_diamonds.lean,scripts/noshake.json 44 n/a ['FR-vdash-bot', 'github-actions', 'grunweg', 'leanprover-bot', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] kbuzzard
assignee:kbuzzard
45-2205
1 month ago
unknown
unknown
24354 grunweg
author:grunweg
chore(HasFiniteIntegral): rename three lemmas Discovered in #24343. --- - [ ] depends on: #24343 (to avoid merge conflicts) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-measure-probability merge-conflict 108/30 Mathlib/MeasureTheory/Function/L1Space/HasFiniteIntegral.lean 1 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
41-7039
1 month ago
41-7040
1 month ago
0-4604
1 hour
13649 FR-vdash-bot
author:FR-vdash-bot
chore: redefine `Nat.div2` `Nat.bodd` The new definitions are faster than the old ones. `Nat.binaryRec` will be moved to batteries (https://github.com/leanprover-community/batteries/pull/799) or core (https://github.com/leanprover/lean4/pull/3756), so relevant contents are moved to a new file temporarily. --- - [x] depends on: #15567 - [x] depends on: #19666 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict 63/88 Mathlib/Computability/Primrec.lean,Mathlib/Data/Int/Bitwise.lean,Mathlib/Data/Nat/Bits.lean,Mathlib/Data/Nat/Bitwise.lean,Mathlib/Data/Nat/Size.lean,Mathlib/Logic/Denumerable.lean,Mathlib/Logic/Encodable/Basic.lean,Mathlib/Logic/Equiv/Nat.lean 8 15 ['FR-vdash-bot', 'digama0', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'urkud'] digama0
assignee:digama0
37-72585
1 month ago
37-72587
1 month ago
87-51692
87 days
14023 mattrobball
author:mattrobball
perf(RingTheory.OreLocalization): make data irreducible We generally do not want to unfold operations passing through `Quotient` if we can avoid it for performance reasons. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict 43/32 Mathlib/GroupTheory/MonoidLocalization.lean,Mathlib/RingTheory/OreLocalization/Basic.lean,Mathlib/RingTheory/OreLocalization/Ring.lean 3 5 ['github-actions', 'grunweg', 'leanprover-bot', 'mattrobball'] nobody
37-44718
1 month ago
345-34541
11 months ago
0-0
0 seconds
4979 mhk119
author:mhk119
doc(Data/Nat/Bitblast): initial commit Initial commit of Bitblast.lean where we prove equivalence of bitblast unsigned less than and bitblast addition. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data merge-conflict 202/4 Mathlib/Data/Bool/Basic.lean,Mathlib/Data/Nat/Bitwise.lean,Mathlib/Data/Nat/Pow.lean 3 49 ['ChrisHughes24', 'digama0', 'goens', 'grunweg', 'j-loreaux', 'kim-em', 'mhk119'] nobody
37-44420
1 month ago
37-44420
1 month ago
7-68358
7 days
24064 kim-em
author:kim-em
chore: replace `norm_num` with `simp` where applicable Consider replacing a tactic with a (ahem) simpler alternative. Fairly neutral performance implications, just depends on whether we would like to encourage people to use `simp` where applicable. merge-conflict 345/345 Archive/Examples/MersennePrimes.lean,Archive/Imo/Imo1959Q2.lean,Archive/Imo/Imo1960Q1.lean,Archive/Imo/Imo1962Q1.lean,Archive/Imo/Imo1962Q4.lean,Archive/Imo/Imo1981Q3.lean,Archive/Imo/Imo1982Q1.lean,Archive/Imo/Imo2001Q2.lean,Archive/Imo/Imo2005Q4.lean,Archive/Imo/Imo2006Q3.lean,Archive/Imo/Imo2008Q4.lean,Archive/Imo/Imo2024Q1.lean,Archive/Imo/Imo2024Q5.lean,Archive/Imo/Imo2024Q6.lean,Archive/Wiedijk100Theorems/AbelRuffini.lean,Archive/Wiedijk100Theorems/CubingACube.lean,Archive/Wiedijk100Theorems/SumOfPrimeReciprocalsDiverges.lean,Counterexamples/Cyclotomic105.lean,Counterexamples/Phillips.lean,Mathlib/Algebra/Field/NegOnePow.lean,Mathlib/Algebra/Homology/HomotopyCategory/MappingCone.lean,Mathlib/Algebra/Order/CauSeq/BigOperators.lean,Mathlib/Algebra/Polynomial/FieldDivision.lean,Mathlib/Algebra/Polynomial/Roots.lean,Mathlib/Algebra/Polynomial/SpecificDegree.lean,Mathlib/Algebra/Ring/BooleanRing.lean,Mathlib/Algebra/Star/CHSH.lean,Mathlib/AlgebraicGeometry/EllipticCurve/IsomOfJ.lean,Mathlib/AlgebraicTopology/DoldKan/Faces.lean,Mathlib/Analysis/Analytic/Inverse.lean,Mathlib/Analysis/Asymptotics/AsymptoticEquivalent.lean,Mathlib/Analysis/BoxIntegral/UnitPartition.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Basic.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Order.lean,Mathlib/Analysis/CStarAlgebra/Module/Defs.lean,Mathlib/Analysis/Calculus/FDeriv/Measurable.lean,Mathlib/Analysis/Calculus/FDeriv/Norm.lean,Mathlib/Analysis/Calculus/FDeriv/Symmetric.lean,Mathlib/Analysis/Complex/AbelLimit.lean,Mathlib/Analysis/Convex/Between.lean,Mathlib/Analysis/Convex/Function.lean,Mathlib/Analysis/Convolution.lean,Mathlib/Analysis/Fourier/AddCircle.lean,Mathlib/Analysis/Fourier/AddCircleMulti.lean,Mathlib/Analysis/Fourier/Inversion.lean,Mathlib/Analysis/Fourier/RiemannLebesgueLemma.lean,Mathlib/Analysis/InnerProductSpace/NormPow.lean,Mathlib/Analysis/InnerProductSpace/Projection.lean,Mathlib/Analysis/InnerProductSpace/l2Space.lean,Mathlib/Analysis/MeanInequalities.lean,Mathlib/Analysis/MellinInversion.lean,Mathlib/Analysis/Normed/Affine/Simplex.lean,Mathlib/Analysis/Normed/Algebra/TrivSqZeroExt.lean,Mathlib/Analysis/Normed/Group/ControlledClosure.lean,Mathlib/Analysis/Normed/Lp/lpSpace.lean,Mathlib/Analysis/Normed/Operator/Banach.lean,Mathlib/Analysis/Normed/Ring/Units.lean,Mathlib/Analysis/NormedSpace/HahnBanach/Separation.lean,Mathlib/Analysis/NormedSpace/MStructure.lean,Mathlib/Analysis/NormedSpace/RieszLemma.lean,Mathlib/Analysis/Oscillation.lean,Mathlib/Analysis/SpecialFunctions/BinaryEntropy.lean,Mathlib/Analysis/SpecialFunctions/Complex/Log.lean,Mathlib/Analysis/SpecialFunctions/ContinuousFunctionalCalculus/Rpow/Basic.lean,Mathlib/Analysis/SpecialFunctions/ContinuousFunctionalCalculus/Rpow/Isometric.lean,Mathlib/Analysis/SpecialFunctions/ExpDeriv.lean,Mathlib/Analysis/SpecialFunctions/Gamma/Beta.lean,Mathlib/Analysis/SpecialFunctions/Gamma/BohrMollerup.lean,Mathlib/Analysis/SpecialFunctions/Gamma/Deligne.lean,Mathlib/Analysis/SpecialFunctions/Gaussian/GaussianIntegral.lean,Mathlib/Analysis/SpecialFunctions/Integrals.lean,Mathlib/Analysis/SpecialFunctions/Log/Monotone.lean,Mathlib/Analysis/SpecialFunctions/Pow/Real.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Angle.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Basic.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Complex.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Inverse.lean,Mathlib/Combinatorics/Additive/AP/Three/Behrend.lean,Mathlib/Combinatorics/Additive/SmallTripling.lean,Mathlib/Combinatorics/Extremal/RuzsaSzemeredi.lean,Mathlib/Combinatorics/SimpleGraph/Density.lean,Mathlib/Combinatorics/SimpleGraph/Regularity/Bound.lean,Mathlib/Combinatorics/SimpleGraph/Regularity/Chunk.lean,Mathlib/Combinatorics/SimpleGraph/Regularity/Increment.lean,Mathlib/Combinatorics/SimpleGraph/Regularity/Lemma.lean,Mathlib/Combinatorics/SimpleGraph/Triangle/Basic.lean,Mathlib/Combinatorics/SimpleGraph/Triangle/Counting.lean,Mathlib/Computability/Ackermann.lean,Mathlib/Computability/AkraBazzi/AkraBazzi.lean,Mathlib/Computability/DFA.lean,Mathlib/Data/Complex/Basic.lean,Mathlib/Data/Complex/Trigonometric.lean,Mathlib/Data/Nat/Bits.lean,Mathlib/Data/Nat/Choose/Central.lean,Mathlib/Data/Nat/Choose/Sum.lean,Mathlib/Data/Nat/Digits.lean,Mathlib/Data/Nat/Prime/Defs.lean,Mathlib/Data/Real/GoldenRatio.lean,Mathlib/Data/Real/Pi/Bounds.lean,Mathlib/Data/Real/Pi/Irrational.lean 171 9 ['github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'leanprover-community-mathlib4-bot'] nobody
37-5710
1 month ago
37-5711
1 month ago
11-65652
11 days
23546 JovanGerb
author:JovanGerb
feat(LinearAlgebra/AffineSpace/AffineSubspace): rename `AffineSubspace.mk'` to `Submodule.shift` In addition to renaming, I've refactored the code a bit: - `mem_mk'_iff_vsub_mem` was obsolete since it was the same as `mem_mk'`, so I removed it (this is due to a change in the definition I made recently) - I added a nonempty instance for `shift` - I added a simp lemma that `shift` isn't equal to `⊥` (the empty affine subspace). I need this for the next point. - Edit: I'll leave this for a later PR. ~I proved a simp lemma that a `shift` is parallel to a `shift` if and only if the linear subspaces are the same.~ - I renamed `mk'_eq` to `shift_direction_eq_self `. - I renamed `eq_or_eq_secondInter_of_mem_mk'_span_singleton_iff_mem` to `eq_or_eq_secondInter_iff_mem_of_mem_shift_span_singleton`. I think it is better to put the `of_mem_mk'_span_singleton` at the end of the name. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-euclidean-geometry merge-conflict 128/99 Mathlib/Algebra/Module/ZLattice/Basic.lean,Mathlib/Geometry/Euclidean/Basic.lean,Mathlib/Geometry/Euclidean/MongePoint.lean,Mathlib/Geometry/Euclidean/PerpBisector.lean,Mathlib/Geometry/Euclidean/Sphere/SecondInter.lean,Mathlib/Geometry/Euclidean/Sphere/Tangent.lean,Mathlib/LinearAlgebra/AffineSpace/AffineSubspace/Defs.lean 7 4 ['JovanGerb', 'github-actions', 'leanprover-community-bot-assistant'] nobody
36-19167
1 month ago
36-19168
1 month ago
26-25420
26 days
24483 Parcly-Taxel
author:Parcly-Taxel
chore: delete >6 month old deprecations (2024-10) See #24271 for the general pattern of regex used in the first (automated) commit. The date range used in this PR is `2024-10-..`. tech debt merge-conflict 2/1182 Mathlib/Algebra/BigOperators/Group/List/Basic.lean,Mathlib/Algebra/CharP/Two.lean,Mathlib/Algebra/Order/Monoid/Unbundled/WithTop.lean,Mathlib/AlgebraicGeometry/Morphisms/ClosedImmersion.lean,Mathlib/AlgebraicGeometry/Morphisms/Preimmersion.lean,Mathlib/AlgebraicGeometry/Restrict.lean,Mathlib/Analysis/Analytic/Basic.lean,Mathlib/Analysis/Calculus/ContDiff/Basic.lean,Mathlib/Analysis/Calculus/ContDiff/Defs.lean,Mathlib/Analysis/Calculus/Deriv/Basic.lean,Mathlib/Analysis/Calculus/Deriv/Comp.lean,Mathlib/Analysis/Calculus/FDeriv/Basic.lean,Mathlib/Analysis/Calculus/FDeriv/Comp.lean,Mathlib/Analysis/Calculus/LineDeriv/Basic.lean,Mathlib/Analysis/Complex/ReImTopology.lean,Mathlib/Analysis/Complex/UpperHalfPlane/Topology.lean,Mathlib/Analysis/LocallyConvex/WeakOperatorTopology.lean,Mathlib/Analysis/LocallyConvex/WithSeminorms.lean,Mathlib/Analysis/Normed/Operator/Banach.lean,Mathlib/Analysis/Normed/Operator/LinearIsometry.lean,Mathlib/Analysis/NormedSpace/OperatorNorm/NormedSpace.lean,Mathlib/CategoryTheory/Limits/Preserves/Limits.lean,Mathlib/CategoryTheory/Sites/Canonical.lean,Mathlib/Data/ENNReal/Inv.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/Data/List/Flatten.lean,Mathlib/Data/List/SplitBy.lean,Mathlib/Data/Nat/Factorization/Basic.lean,Mathlib/Data/Nat/Factorization/Defs.lean,Mathlib/Data/Nat/Factorization/PrimePow.lean,Mathlib/Data/Set/Subset.lean,Mathlib/FieldTheory/IntermediateField/Adjoin/Algebra.lean,Mathlib/Geometry/Manifold/ContMDiff/Defs.lean,Mathlib/Geometry/Manifold/LocalInvariantProperties.lean,Mathlib/Geometry/Manifold/MFDeriv/Basic.lean,Mathlib/GroupTheory/CosetCover.lean,Mathlib/GroupTheory/GroupAction/Blocks.lean,Mathlib/LinearAlgebra/Eigenspace/Basic.lean,Mathlib/MeasureTheory/Constructions/BorelSpace/Basic.lean,Mathlib/MeasureTheory/Function/StronglyMeasurable/AEStronglyMeasurable.lean,Mathlib/MeasureTheory/Measure/DiracProba.lean,Mathlib/MeasureTheory/Measure/FiniteMeasure.lean,Mathlib/MeasureTheory/Measure/ProbabilityMeasure.lean,Mathlib/NumberTheory/NumberField/Embeddings.lean,Mathlib/Order/InitialSeg.lean,Mathlib/Order/WellFounded.lean,Mathlib/Probability/Density.lean,Mathlib/RingTheory/Finiteness/Cardinality.lean,Mathlib/RingTheory/Finiteness/Ideal.lean,Mathlib/RingTheory/Jacobson/Ring.lean,Mathlib/RingTheory/Localization/Cardinality.lean,Mathlib/RingTheory/PowerSeries/Basic.lean,Mathlib/RingTheory/Spectrum/Prime/TensorProduct.lean,Mathlib/RingTheory/Spectrum/Prime/Topology.lean,Mathlib/SetTheory/Game/Nim.lean,Mathlib/SetTheory/PGame/Algebra.lean,Mathlib/Tactic/FunProp/ContDiff.lean,Mathlib/Topology/AlexandrovDiscrete.lean,Mathlib/Topology/Algebra/ConstMulAction.lean,Mathlib/Topology/Algebra/Constructions.lean,Mathlib/Topology/Algebra/Constructions/DomMulAct.lean,Mathlib/Topology/Algebra/Group/Basic.lean,Mathlib/Topology/Algebra/Group/CompactOpen.lean,Mathlib/Topology/Algebra/Group/Quotient.lean,Mathlib/Topology/Algebra/GroupWithZero.lean,Mathlib/Topology/Algebra/InfiniteSum/Basic.lean,Mathlib/Topology/Algebra/Module/Alternating/Topology.lean,Mathlib/Topology/Algebra/Module/Equiv.lean,Mathlib/Topology/Algebra/Module/Multilinear/Topology.lean,Mathlib/Topology/Algebra/Module/StrongTopology.lean,Mathlib/Topology/Algebra/Module/WeakBilin.lean,Mathlib/Topology/Algebra/Monoid.lean,Mathlib/Topology/Algebra/MulAction.lean,Mathlib/Topology/Algebra/Ring/Ideal.lean,Mathlib/Topology/Algebra/SeparationQuotient/Section.lean,Mathlib/Topology/Algebra/StarSubalgebra.lean,Mathlib/Topology/Bases.lean,Mathlib/Topology/Category/Profinite/Nobeling/Induction.lean,Mathlib/Topology/Category/TopCat/EffectiveEpi.lean,Mathlib/Topology/Category/TopCat/Limits/Products.lean,Mathlib/Topology/Category/TopCat/Limits/Pullbacks.lean,Mathlib/Topology/Clopen.lean,Mathlib/Topology/CompactOpen.lean,Mathlib/Topology/Compactness/Compact.lean,Mathlib/Topology/Compactness/Lindelof.lean,Mathlib/Topology/Compactness/LocallyCompact.lean,Mathlib/Topology/Compactness/SigmaCompact.lean,Mathlib/Topology/Connected/Basic.lean,Mathlib/Topology/Connected/Clopen.lean,Mathlib/Topology/Connected/PathConnected.lean,Mathlib/Topology/Connected/TotallyDisconnected.lean,Mathlib/Topology/Constructions.lean,Mathlib/Topology/Constructions/SumProd.lean,Mathlib/Topology/ContinuousMap/Bounded/Basic.lean,Mathlib/Topology/ContinuousMap/ContinuousMapZero.lean,Mathlib/Topology/ContinuousMap/Sigma.lean,Mathlib/Topology/ContinuousMap/T0Sierpinski.lean,Mathlib/Topology/ContinuousOn.lean,Mathlib/Topology/Covering.lean,Mathlib/Topology/Defs/Induced.lean 139 3 ['github-actions', 'leanprover-community-bot-assistant'] nobody
35-41124
1 month ago
35-41126
1 month ago
4-54091
4 days
21751 vihdzp
author:vihdzp
refactor(SetTheory/Ordinal/Arithmetic): rework `Ordinal.pred` API This PR does the following: - give a simpler definition of `Ordinal.pred` - replace `¬ ∃ a, o = succ a` and `∀ a, o ≠ succ a` by `IsSuccPrelimit o` throughout - improve theorem names --- There's a legitimate question of whether we even want `Ordinal.pred` (see [Zulip](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Ordinal.2Epred)) but this should be a good change in the meanwhile regardless. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-set-theory maintainer-merge merge-conflict 102/67 Mathlib/SetTheory/Ordinal/Arithmetic.lean,Mathlib/SetTheory/Ordinal/Exponential.lean 2 13 ['YaelDillies', 'github-actions', 'grunweg', 'vihdzp'] nobody
33-79798
1 month ago
80-58425
2 months ago
36-50134
36 days
9273 grunweg
author:grunweg
feat: extended charts are local diffeomorphisms on their source --- TODO: I think this should hold at any interior point - as the inverse of the extended chart, restricted to the interior of its source, will be a local inverse. The analogous result for un-extended charts is shown in #8160. Unresolved questions - are all the tiny API lemmas useful; are any more missing? - do I want similar results for `extChartAt`? (In any case, they are easy to deduce.) - [ ] depends on: #8738 for simplicity [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-differential-geometry merge-conflict 225/12 Mathlib/Geometry/Manifold/ContMDiff/Atlas.lean,Mathlib/Geometry/Manifold/LocalDiffeomorph.lean,Mathlib/Topology/Algebra/Module/Basic.lean 3 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
31-80975
1 month ago
unknown
unknown
19985 vihdzp
author:vihdzp
feat(SetTheory/ZFC/Ordinal): Lean ordinals to ZFC ordinals We define `Ordinal.toZFSet` and prove that its outputs are precisely the ZFC ordinals. --- - [ ] depends on: #19946 - [x] depends on: #19970 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-set-theory merge-conflict 208/6 Mathlib/Order/SuccPred/CompleteLinearOrder.lean,Mathlib/SetTheory/ZFC/Basic.lean,Mathlib/SetTheory/ZFC/Ordinal.lean,Mathlib/SetTheory/ZFC/Rank.lean 4 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
31-13249
1 month ago
31-13252
1 month ago
0-562
9 minutes
17027 vihdzp
author:vihdzp
feat(SetTheory/ZFC/Ordinal): von Neumann hierarchy of sets --- - [x] depends on: #16996 - [x] depends on: #17016 - [x] depends on: #17026 - [x] depends on: #18239 - [ ] depends on: #19946 - [x] depends on: #19967 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-set-theory merge-conflict 204/29 Mathlib.lean,Mathlib/SetTheory/Ordinal/Basic.lean,Mathlib/SetTheory/ZFC/Basic.lean,Mathlib/SetTheory/ZFC/Neumann.lean,Mathlib/SetTheory/ZFC/Rank.lean 5 8 ['alreadydone', 'github-actions', 'mathlib4-dependent-issues-bot', 'vihdzp'] nobody
31-13200
1 month ago
31-13202
1 month ago
0-344
5 minutes
23338 WilliamCoram
author:WilliamCoram
feat: restricted power series form a ring We define restricted powerseries over a normed ring R, and show they form a ring when R has the ultrametric property. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-number-theory merge-conflict 186/0 Mathlib.lean,Mathlib/RingTheory/PowerSeries/Restricted.lean 2 18 ['Paul-Lez', 'WilliamCoram', 'github-actions', 'grunweg', 'leanprover-community-bot-assistant'] nobody
26-33783
26 days ago
26-33785
26 days ago
48-76736
48 days
24590 smmercuri
author:smmercuri
chore: make `Valuation.Completion` a `def` and refactor more of `AdicValuation.lean` The main purpose of this PR is to resolve timeout issues encountered in FLT following the refactor of `HeightOneSpectrum.adicCompletion` to use the `WithVal` type synonym. The proposed fix in this PR is to replace `abbrev` with `def` in `Valuation.Completion`. Tested in FLT and this removes the timeout issue. Also refactor as much API as possible from `HeightOneSpectrum.adicCompletion` to `Valuation.Completion`. See #22488 for a previous attempt at fixing the problem. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) FLT merge-conflict 162/81 Mathlib/NumberTheory/NumberField/FinitePlaces.lean,Mathlib/RingTheory/DedekindDomain/AdicValuation.lean,Mathlib/RingTheory/DedekindDomain/FiniteAdeleRing.lean,Mathlib/RingTheory/LaurentSeries.lean,Mathlib/Topology/Algebra/Valued/WithVal.lean 5 5 ['github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'smmercuri'] nobody
22-78761
22 days ago
22-78763
22 days ago
13-35725
13 days
24245 JovanGerb
author:JovanGerb
feat(Geometry/Euclidean/SignedDist): `signedDist` between two points This PR defines `signedDist`, the signed distance between two points. It redefines `signedInfDist` so that it uses `signedDist`. The motivation is to use this in IMO2020Q6. Additionally this definition will be useful for properly reasoning about the power of a point [#mathlib4 > Signed distance between points](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Signed.20distance.20between.20points) some comments: * should `signedDistLinear` be `private`? * should `signedDist` and `signedInfDist` be made continuous bunled maps in this PR? * I'm not too happy about the hypothesis in `signedDist_congr (h : ∃ r > (0 : ℝ), r • v = w)`. This relationship between `v` and `w` is a symmetric one that should have some API around it, similar to `SameRay`. It could also be spelled as `(ℝ≥0 ∙ v) = ℝ≥0 ∙ w` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-euclidean-geometry merge-conflict 206/23 Mathlib/Analysis/InnerProductSpace/Basic.lean,Mathlib/Geometry/Euclidean/SignedDist.lean,Mathlib/Topology/MetricSpace/Pseudo/Defs.lean 3 2 ['github-actions', 'leanprover-community-bot-assistant'] nobody
18-84326
18 days ago
18-84328
18 days ago
30-61949
30 days
22837 joneugster
author:joneugster
feat(Data/Set/Basic): add subset_iff and not_mem_subset_iff Add `Set.subset_iff` for consistent API with `Finset.subset_iff`. Add `Set.not_mem_subset_iff` and `Finset.not_mem_subset_iff`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-set-theory t-data merge-conflict 9/0 Mathlib/Data/Finset/Defs.lean,Mathlib/Data/Set/Basic.lean 2 4 ['Ruben-VandeVelde', 'github-actions', 'joneugster', 'leanprover-community-bot-assistant'] nobody
15-22167
15 days ago
15-22169
15 days ago
30-35190
30 days
21476 grunweg
author:grunweg
feat(lint-style): enable running on downstream projects Enable lint-style to run on downstream projects, by making the following modifications: - allow passing an explicit list of libraries to lint: if nothing is passed, it lints `Mathlib`, `Archive` and `Counterexamples` (as before); otherwise, it lints precisely the passed modules - only check init imports, undocumented scripts and the errors from `lint-style.py` when linting Mathlib - make the style exceptions file configurable and optional: using the `nolints-file` flag, the exceptions file can be configured. If the flag is omitted, we try to find a file at `scripts/nolints-style.txt` --- and otherwise proceed with no style exceptions. This means mathlib can continue unchanged, and downstream projects can either add an explicit exceptions file, or proceed without any exceptions. After this PR, one should be able to run lint-style on a downstream project by `lake exe lint-style ProjectName`. Prompted by [this zulip discussion](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/lint-style.20for.20downstream.20libraries). --- - [ ] depends on: #24570 - [ ] depends on: #24953 (I did not test the last part.) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-linter merge-conflict 58/19 Mathlib/Tactic/Linter/TextBased.lean,scripts/lint-style.lean 2 19 ['Vierkantor', 'adomani', 'github-actions', 'grunweg', 'joneugster', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] joneugster
assignee:joneugster
14-27655
14 days ago
14-27658
14 days ago
43-17409
43 days
23349 BGuillemet
author:BGuillemet
feat: add LocallyLipschitzOn.lipschitzOnWith_of_isCompact and two small lemmas about Lipschitz functions Main feat (in Mathlib/Topology/EMetricSpace/Basic.lean): if a function `f` from an extended pseudometric space to a pseudometric space is locally Lipschitz on a compact subset `s`, then `f` is Lipschitz on `s`. The theorem is true only when the codomain of `f` is a pseudometric space, so it needs imports from Mathlib/Topology/MetricSpace. Other small feat (in Mathlib/Analysis/Calculus/ContDiff/RCLike.lean): a function that is continuously differentiable on an open subset is locally Lipschitz on this subset. --- - [ ] depends on: #22890 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import new-contributor t-topology merge-conflict 59/4 Mathlib/Analysis/Calculus/ContDiff/RCLike.lean,Mathlib/Topology/EMetricSpace/Lipschitz.lean 2 4 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] PatrickMassot
assignee:PatrickMassot
13-9385
13 days ago
13-9387
13 days ago
35-30364
35 days
23333 mariainesdff
author:mariainesdff
feat(Analysis.Normed.Unbundled.SpectralNormUnique): prove unique extension theorem Let `K` be a field complete with respect to a nontrivial nonarchimedean multiplicative norm and `L/K` be an algebraic extension. We show that the spectral norm on `L` is a nonarchimedean multiplicative norm, and any power-multiplicative `K`-algebra norm on `L` coincides with the spectral norm. More over, if `L/K` is finite, then `L` is a complete space. This result is [S. Bosch, U. Güntzer, R. Remmert,*Non-Archimedean Analysis* (Theorem 3.2.4/2)][bosch-guntzer-remmert]. --- - [ ] depends on: #23301 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-analysis t-number-theory merge-conflict 1487/3 Mathlib.lean,Mathlib/Algebra/Order/BigOperators/Ring/Finset.lean,Mathlib/Algebra/Order/BigOperators/Ring/Multiset.lean,Mathlib/Algebra/Polynomial/Basic.lean,Mathlib/Algebra/Polynomial/BigOperators.lean,Mathlib/Algebra/Polynomial/Lifts.lean,Mathlib/Algebra/Polynomial/RingDivision.lean,Mathlib/Algebra/Polynomial/Splits.lean,Mathlib/Analysis/Normed/Unbundled/AlgNormOfGalois.lean,Mathlib/Analysis/Normed/Unbundled/RingSeminorm.lean,Mathlib/Analysis/Normed/Unbundled/SpectralNorm.lean,Mathlib/Analysis/Normed/Unbundled/SpectralNormUnique.lean,Mathlib/Data/Finset/Max.lean,Mathlib/Data/List/MinMax.lean,Mathlib/Data/NNReal/Basic.lean,Mathlib/Data/Real/IsNonarchimedean.lean,Mathlib/Data/Real/Pointwise.lean,Mathlib/FieldTheory/IntermediateField/Adjoin/Basic.lean,Mathlib/FieldTheory/IsAlgClosed/AlgebraicClosure.lean,Mathlib/Order/ConditionallyCompleteLattice/Finset.lean,Mathlib/Order/ConditionallyCompleteLattice/Indexed.lean 21 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
12-77352
12 days ago
12-77354
12 days ago
0-0
0 seconds
23767 grunweg
author:grunweg
refactor: make library notes a definition Make library notes a definition of `Unit` type, whose doc-string is the note's content. As a consequence, - doc-gen will display all library notes without any custom logic, - library notes are shown upon hover (via the use of the doc-string), - go do definition for library notes is easy Automate this using a macro, which also enforces that all library notes are inside the Mathlib.LibraryNote namespace. *Temporarily*, we use the `library_note2` name; if/when the batteries version is changed, we can reclaim the original name. This PR does not address how to *refer* to library notes nicely (in a way that is shown in the documentation, checked for typos, with sufficient imports ensured etc.). That is left to a future PR. This is proposal 2a from this [zulip discussion]([#mathlib4 > library notes @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/library.20notes/near/510614740)) ------------ Open questions/TODOs: - should this go in batteries instead? can the old definition just be overwritten? - otherwise, what's the best place for the `LibraryNote` definition? A single file just for this feels overkill; I put it in Mathlib.Tactic.Basic for now. I could use Mathlib.Init, of course (but that might be excessive) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-meta merge-conflict 48/48 Archive/Imo/Imo2019Q2.lean,Mathlib/Algebra/BigOperators/Group/Finset/Defs.lean,Mathlib/Algebra/Category/Ring/Limits.lean,Mathlib/Algebra/Group/Action/Defs.lean,Mathlib/Algebra/Group/Conj.lean,Mathlib/Algebra/Group/Defs.lean,Mathlib/Algebra/Group/Hom/Defs.lean,Mathlib/Algebra/Group/Pointwise/Set/Basic.lean,Mathlib/Algebra/Group/Pointwise/Set/Scalar.lean,Mathlib/Algebra/Group/Submonoid/Operations.lean,Mathlib/Algebra/HierarchyDesign.lean,Mathlib/Algebra/Order/Hom/Basic.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Note.lean,Mathlib/Analysis/RCLike/Lemmas.lean,Mathlib/CategoryTheory/Category/Basic.lean,Mathlib/Data/NNRat/Defs.lean,Mathlib/Data/Nat/Cast/Defs.lean,Mathlib/Data/Nat/Init.lean,Mathlib/Geometry/Manifold/Algebra/Monoid.lean,Mathlib/Geometry/Manifold/ChartedSpace.lean,Mathlib/Logic/Basic.lean,Mathlib/Tactic/Basic.lean,Mathlib/Tactic/NormNum/Basic.lean,Mathlib/Tactic/Simps/Basic.lean,Mathlib/Topology/Algebra/Nonarchimedean/Bases.lean,Mathlib/Topology/Continuous.lean 26 9 ['adomani', 'github-actions', 'grunweg', 'leanprover-community-bot-assistant'] nobody
11-22480
11 days ago
11-22482
11 days ago
51-69759
51 days
21129 chrisflav
author:chrisflav
perf(RingTheory/Kaehler/JacobiZariski): reorder universe variables Naming of universe variables has an impact on universe unification. It seems to matter that the universe variables of `R`, `S` and `T` appear before the universe variables of the generators in alphabetical order. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) performance-hack t-algebra merge-conflict
label:t-algebra$
18/20 Mathlib/RingTheory/Kaehler/JacobiZariski.lean 1 38 ['chrisflav', 'erdOne', 'github-actions', 'grunweg', 'kbuzzard', 'leanprover-bot', 'leanprover-community-bot-assistant', 'mattrobball'] nobody
7-24653
7 days ago
7-24655
7 days ago
125-81208
125 days
25138 chrisflav
author:chrisflav
chore(RingTheory): remove unnecessary `toRingHom` coercions --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict
label:t-algebra$
32/40 Mathlib/RingTheory/Extension/Presentation/Basic.lean,Mathlib/RingTheory/FinitePresentation.lean,Mathlib/RingTheory/Ideal/Cotangent.lean,Mathlib/RingTheory/Ideal/Maps.lean,Mathlib/RingTheory/Ideal/Quotient/Operations.lean,Mathlib/RingTheory/Smooth/Basic.lean,Mathlib/RingTheory/Smooth/Kaehler.lean,Mathlib/RingTheory/Spectrum/Prime/ChevalleyComplexity.lean,Mathlib/RingTheory/Unramified/Basic.lean 9 5 ['chrisflav', 'erdOne', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant'] nobody
7-10781
7 days ago
7-10783
7 days ago
9-64502
9 days
21182 joneugster
author:joneugster
fix(Util/CountHeartbeats): move elaboration in #count_heartbeats inside a namespace Currently the `#count_heartbeat` linter reported the heartbeats until it concluded `error: [declaration] has already been declared` instead of re-elaborating the declaration. --- [Zulip report](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/count_heartbeats.20for.20all.20declarations.20in.20a.20file.3F/near/496303652) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta merge-conflict 72/5 Mathlib/Util/CountHeartbeats.lean,MathlibTest/CountHeartbeats.lean 2 17 ['adomani', 'github-actions', 'joneugster', 'leanprover-community-bot-assistant', 'mathlib-bors'] adomani
assignee:adomani
6-38133
6 days ago
6-38134
6 days ago
64-19141
64 days
24877 smmercuri
author:smmercuri
feat: predicates for extensions of complex embeddings If `L/K`, `ψ : K →+* ℂ`, `φ : L →+* ℂ` we define three predicates asserting ways that `φ` can extend `ψ`. - `IsExtension ψ φ` : the restriction of `φ` to `K` is `ψ`. - `IsMixedExtension ψ φ` : the restriction of `φ` to `K` is `ψ`, `ψ` has real image while `φ` has complex image. - `IsUnmixedExtension ψ φ`: the restriction of `φ` to `K` is `ψ`, `ψ` has real image if and only if `φ` has real image. `IsMixedExtension` and `IsUnmixedExtension` are the `ComplexEmbedding` analogues to ramified and unramified infinite places. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-number-theory merge-conflict 91/0 Mathlib/NumberTheory/NumberField/InfinitePlace/Embeddings.lean 1 7 ['github-actions', 'leanprover-community-bot-assistant', 'smmercuri', 'xroblot'] nobody
5-7757
5 days ago
5-7759
5 days ago
21-40253
21 days
7596 alreadydone
author:alreadydone
feat: covering maps from properly discontinuous actions and discrete subgroups --- - [x] depends on: #23236 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) file-removed t-topology merge-conflict 351/21 Mathlib.lean,Mathlib/Analysis/SpecialFunctions/Complex/Circle.lean,Mathlib/Topology/Algebra/ConstMulAction.lean,Mathlib/Topology/Algebra/Group/Pointwise.lean,Mathlib/Topology/Covering/AddCircle.lean,Mathlib/Topology/Covering/Basic.lean,Mathlib/Topology/Covering/Galois.lean,Mathlib/Topology/Homotopy/Lifting.lean,Mathlib/Topology/Instances/AddCircle.lean 9 17 ['ADedecker', 'alreadydone', 'digama0', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'tb65536'] nobody
3-27315
3 days ago
3-27317
3 days ago
48-80629
48 days
25340 dupuisf
author:dupuisf
chore(Analysis/Convex): move files pertaining to convex/concave functions to their own folder This PR creates a new folder under `Analysis/Convex` called `Analysis/Convex/Function`, which includes files that are mostly or entirely about convex/concave functions (as opposed to convex sets). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-convex-geometry merge-conflict 4264/4155 Mathlib.lean,Mathlib/Analysis/Convex/Continuous.lean,Mathlib/Analysis/Convex/Deriv.lean,Mathlib/Analysis/Convex/Exposed.lean,Mathlib/Analysis/Convex/Extrema.lean,Mathlib/Analysis/Convex/Function.lean,Mathlib/Analysis/Convex/Function/Basic.lean,Mathlib/Analysis/Convex/Function/Continuous.lean,Mathlib/Analysis/Convex/Function/Deriv.lean,Mathlib/Analysis/Convex/Function/Extrema.lean,Mathlib/Analysis/Convex/Function/Integral.lean,Mathlib/Analysis/Convex/Function/Jensen.lean,Mathlib/Analysis/Convex/Function/Mul.lean,Mathlib/Analysis/Convex/Function/Piecewise.lean,Mathlib/Analysis/Convex/Function/Quasiconvex.lean,Mathlib/Analysis/Convex/Function/Slope.lean,Mathlib/Analysis/Convex/Function/Strong.lean,Mathlib/Analysis/Convex/Integral.lean,Mathlib/Analysis/Convex/Jensen.lean,Mathlib/Analysis/Convex/Mul.lean,Mathlib/Analysis/Convex/Piecewise.lean,Mathlib/Analysis/Convex/Quasiconvex.lean,Mathlib/Analysis/Convex/Slope.lean,Mathlib/Analysis/Convex/SpecificFunctions/Basic.lean,Mathlib/Analysis/Convex/SpecificFunctions/Deriv.lean,Mathlib/Analysis/Convex/Strong.lean,Mathlib/Analysis/MeanInequalities.lean,Mathlib/Analysis/MeanInequalitiesPow.lean,Mathlib/Analysis/Normed/Module/Convex.lean,Mathlib/Analysis/Seminorm.lean,Mathlib/Analysis/SpecialFunctions/Log/NegMulLog.lean,Mathlib/Analysis/SpecialFunctions/Pochhammer.lean,Mathlib/MeasureTheory/Measure/Decomposition/IntegralRNDeriv.lean,Mathlib/NumberTheory/Harmonic/GammaDeriv.lean 34 2 ['github-actions', 'leanprover-community-bot-assistant'] nobody
2-32212
2 days ago
2-32214
2 days ago
6-40169
6 days
25012 urkud
author:urkud
refactor(*): migrate from `Matrix.toLin'` to `Matrix.mulVecLin` or `Matrix.mulVec` whenever we don't need the `LinearEquiv.symm` part. See [Zulip discussion](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Matrix.2EtoLin'.20vs.20Matrix.2EmulVecLin/with/515188548). It makes sense to have only one normal form, and `Matrix.toLin'` has an extra `DecidableEq` assumption. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict 154/122 Mathlib/Algebra/Lie/Matrix.lean,Mathlib/Algebra/Module/Equiv/Basic.lean,Mathlib/Analysis/CStarAlgebra/Matrix.lean,Mathlib/Analysis/Matrix.lean,Mathlib/Combinatorics/SimpleGraph/LapMatrix.lean,Mathlib/Data/Matrix/Rank.lean,Mathlib/LinearAlgebra/Basis/Defs.lean,Mathlib/LinearAlgebra/Determinant.lean,Mathlib/LinearAlgebra/Finsupp/VectorSpace.lean,Mathlib/LinearAlgebra/FreeModule/Finite/Matrix.lean,Mathlib/LinearAlgebra/Matrix/BilinearForm.lean,Mathlib/LinearAlgebra/Matrix/Charpoly/Minpoly.lean,Mathlib/LinearAlgebra/Matrix/Diagonal.lean,Mathlib/LinearAlgebra/Matrix/Gershgorin.lean,Mathlib/LinearAlgebra/Matrix/SesquilinearForm.lean,Mathlib/LinearAlgebra/Matrix/SpecialLinearGroup.lean,Mathlib/LinearAlgebra/Matrix/ToLin.lean,Mathlib/LinearAlgebra/Matrix/ToLinearEquiv.lean,Mathlib/LinearAlgebra/UnitaryGroup.lean,Mathlib/MeasureTheory/Measure/Lebesgue/Basic.lean,Mathlib/RingTheory/Smooth/StandardSmooth.lean 21 3 ['github-actions', 'leanprover-community-bot-assistant'] nobody
1-27046
1 day ago
1-27048
1 day ago
15-74981
15 days
23394 BoltonBailey
author:BoltonBailey
chore(Data/Int/WithZero): fix erw --- Removing an `erw`. This is my first time doing this, so please tell me if I am doing something wrong here (e.g. should the new lemma be `simp`?). [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) tech debt merge-conflict 5/4 Mathlib/Algebra/Group/WithOne/Defs.lean,Mathlib/Algebra/GroupWithZero/WithZero.lean,Mathlib/Data/Int/WithZero.lean 3 19 ['BoltonBailey', 'Ruben-VandeVelde', 'eric-wieser', 'fpvandoorn', 'github-actions', 'grunweg', 'leanprover-community-bot-assistant'] nobody
0-50895
14 hours ago
0-50897
14 hours ago
52-38111
52 days
25264 linesthatinterlace
author:linesthatinterlace
feat: add elementary lifts for `OneHom`, `MulHom`, `MonoidHom` and `RingHom`. Adds `liftRight` and `liftLeft` constructions for `OneHom`, `MulHom` and `MonoidHom`. --- The plan is to implement `Units.liftRight` and possibly other "lift"-style monoid constructions (e.g. `liftOfRightInverse`) using these. This should probably be in a future PR but I could consider adding it to this one once the initial changes are stable. Note that these constructions are added relatively deep as they do not need much in the way of pre-requisites. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict
label:t-algebra$
412/11 Mathlib/Algebra/Group/Hom/Basic.lean,Mathlib/Algebra/Group/Hom/Defs.lean,Mathlib/Algebra/Ring/Hom/Basic.lean,Mathlib/Algebra/Ring/Hom/Defs.lean 4 7 ['eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'linesthatinterlace'] nobody
0-5787
1 hour ago
0-5789
1 hour ago
12-4669
12 days

Stale new contributor PRs

Number Author Title Description Labels +/- Modified files (first 100) 📝 💬 All users who commented or reviewed Assignee(s) Updated Last status change total time in review
15224 AnthonyBordg
author:AnthonyBordg
feat(CategoryTheory/Sites): covering families and their associated Grothendieck topology Define covering families on a category and their associated Grothendieck topology by using the API for `Coverage`. Give an explicit characterization of the covering sieves of the said topology. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-category-theory awaiting-author 112/0 Mathlib.lean,Mathlib/CategoryTheory/Sites/CoveringFamilies.lean 2 20 ['AnthonyBordg', 'adamtopaz', 'dagurtomas', 'github-actions', 'joelriou'] nobody
308-17782
10 months ago
313-11447
10 months ago
1-48443
1 day
14563 awueth
author:awueth
feat: if-then-else of exclusive or statement --- If `¬(P ∧ Q)` then `ite (P ∨ Q) a 1 = (ite P a 1) * (ite Q a 1)` [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra awaiting-author
label:t-algebra$
5/0 Mathlib/Algebra/Group/Basic.lean 1 3 ['eric-wieser', 'github-actions', 'kim-em'] nobody
298-35158
9 months ago
298-35158
9 months ago
6-38745
6 days
11207 luigi-massacci
author:luigi-massacci
feat(Topology/MetricSpace): Add new file with type of Katetov maps add a type of Katetov maps (one point extensions of a metric) and related notation and FunLike coercions. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-topology WIP 138/0 Mathlib.lean,Mathlib/Topology/MetricSpace/Katetov.lean,docs/references.bib 3 16 ['fpvandoorn', 'jcommelin', 'kim-em', 'luigi-massacci', 'urkud'] nobody
294-19535
9 months ago
396-21620
1 year ago
26-83567
26 days
11090 pangelinos
author:pangelinos
feat: define spectral spaces and prove that a quasi-compact open of a spectral space is spectral Define spectral spaces and prove that a quasi-compact open of a spectral space is spectral. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-topology please-adopt good first issue 69/0 Topology/Spectral/basic.lean 1 15 ['YaelDillies', 'adomani', 'j-loreaux', 'jcommelin', 'kim-em', 'pangelinos'] nobody
294-19410
9 months ago
298-32336
9 months ago
16-44803
16 days
15121 Eloitor
author:Eloitor
feat: iff theorems for IsSplitEpi and IsSplitMono in opposite category --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-category-theory awaiting-author 40/0 Mathlib/CategoryTheory/EpiMono.lean 1 3 ['github-actions', 'joelriou', 'mattrobball'] nobody
280-81302
9 months ago
312-40561
10 months ago
7-3203
7 days
16773 arulandu
author:arulandu
feat(Probability/Distributions): formalize Beta distribution Formalize Beta distribution, using Gamma distribution as a reference. Added real-valued beta wrapper, in the manner of gamma. Thanks to @EtienneC30 for help with casting real <-> complex. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-measure-probability awaiting-author 286/1 Mathlib.lean,Mathlib/Analysis/SpecialFunctions/Gamma/Beta.lean,Mathlib/Probability/Distributions/Beta.lean 3 48 ['EtienneC30', 'arulandu', 'github-actions', 'vihdzp'] arulandu
assignee:arulandu
262-41519
8 months ago
267-38237
8 months ago
1-21124
1 day
14237 js2357
author:js2357
feat: Define the localization of a fractional ideal at a prime ideal Define the localization of a fractional ideal at a prime ideal, and prove some basic properties. --- This PR is part 3 out of 4 of a proof of `isDedekindDomain_iff_isDedekindDomainDvr`. Part 4 is available here: #14242 - [x] depends on: #14099 Part 1 - [x] depends on: #14216 Part 2 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra awaiting-author
label:t-algebra$
230/0 Mathlib.lean,Mathlib/RingTheory/FractionalIdeal/LocalizedAtPrime.lean,Mathlib/RingTheory/Localization/Basic.lean 3 20 ['Vierkantor', 'YaelDillies', 'github-actions', 'js2357', 'kbuzzard', 'leanprover-community-mathlib4-bot'] Vierkantor
assignee:Vierkantor
258-20363
8 months ago
258-20481
8 months ago
26-39463
26 days
14603 awueth
author:awueth
feat: degree is invariant under graph isomorphism --- Mathlib has the definition `SimpleGraph.Iso.mapNeighborSet` which is an equivalence between neighbor sets induced by an isomorphism. Would it be beneficial to add the same equivalence for `neighborFinset`? [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-combinatorics WIP 24/0 Mathlib/Combinatorics/SimpleGraph/Map/Finite.lean 1 11 ['awueth', 'github-actions', 'jcommelin', 'kim-em', 'urkud'] nobody
230-13904
7 months ago
230-13904
7 months ago
31-44440
31 days
15809 archiebrowne
author:archiebrowne
feat(RingTheory/MvPolynomial/Ideal): introduce new lemmas about MvPolynomial Ideals Four new lemmas about MvPolynomialIdeals `sub_span_span_sub`, `span_eq_iff_basis_sub`, `mem_basis_mem_span`, `mem_span_exists_dvd_mem_basis`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra awaiting-author
label:t-algebra$
38/0 Mathlib/RingTheory/MvPolynomial/Ideal.lean 1 6 ['Ruben-VandeVelde', 'github-actions', 'riccardobrasca'] riccardobrasca
assignee:riccardobrasca
203-16688
6 months ago
258-18608
8 months ago
41-7533
41 days
20029 FrederickPu
author:FrederickPu
Allow for Config attributes to be set directly Allow for Config attributes to be set directly when using initialize_simp_projection as per issue #19895 Basically modified initialize_simp_projection so that the user has the option of specifying a tuple of config option values. Ex: ``` initialize_simp_projection MulEquiv (toFun → apply, invFun → symm_apply) (fullyApplied := false) ``` These config options are then converted into projections.  --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-meta WIP 34/4 Mathlib/Tactic/Simps/Basic.lean 1 10 ['FrederickPu', 'YaelDillies', 'fpvandoorn', 'github-actions'] nobody
172-85146
5 months ago
173-33855
5 months ago
0-34081
9 hours
18461 hannahfechtner
author:hannahfechtner
feat: left and right common multiples mixins add mixins for left and right common multiples. These carry the data of what factors are used to create the common multiples --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra awaiting-author
label:t-algebra$
78/0 Mathlib/Algebra/Group/Defs.lean 1 13 ['github-actions', 'hannahfechtner', 'jcommelin', 'kbuzzard', 'kim-em', 'trivial1711'] nobody
140-38439
4 months ago
140-38439
4 months ago
69-35596
69 days
20797 vbeffara
author:vbeffara
feat(Topology/Covering): CM version of eq_of_comp_eq Add equivalents of the lemmas `IsCoveringMap.eq_of_comp_eq` and `IsCoveringMap.const_of_comp_CM` for the case of bundled `ContinuousMap` parameters. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-topology easy awaiting-author 9/1 Mathlib/Topology/Covering.lean 1 4 ['github-actions', 'ocfnash', 'vbeffara'] nobody
140-25204
4 months ago
141-26157
4 months ago
2-77310
2 days
19582 yu-yama
author:yu-yama
feat(GroupExtension/Abelian): define `OfMulDistribMulAction.equivH2` Mainly defines: - `structure GroupExtension.OfMulDistribMulAction N G [MulDistribMulAction G N]`: group extensions of `G` by `N` where the multiplicative action of `G` on `N` is the conjugation - `structure GroupExtension.OfMulDistribMulActionWithSection N G [MulDistribMulAction G N]`: group extensions with specific choices of sections - `def GroupExtension.OfMulDistribMulAction.equivH2`: a bijection between the equivalence classes of group extensions and $H^2 (G, N)$ - [x] depends on: #20802 (split PR: contains changes to the `Defs` file) - [x] depends on: #20998 (split PR: mainly adds the `Basic` file) - [ ] depends on: #21837 (split PR: adds the first part of the `Abelian` file) --- Here is a relevant TODO in Mathlib: https://github.com/leanprover-community/mathlib4/blob/4e9fa40d7c480937e09cd6e47a591bd6f3b8be42/Mathlib/RepresentationTheory/GroupCohomology/LowDegree.lean#L46-L48 I would appreciate your comments. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra blocked-by-other-PR
label:t-algebra$
736/14 Mathlib.lean,Mathlib/GroupTheory/GroupExtension/Abelian.lean,Mathlib/GroupTheory/GroupExtension/Defs.lean,docs/references.bib 4 3 ['erdOne', 'github-actions', 'mathlib4-dependent-issues-bot'] nobody
116-3145
3 months ago
116-6919
3 months ago
43-23183
43 days
13442 dignissimus
author:dignissimus
feat: mabel tactic for multiplicative abelian groups Mabel tactic for multiplicative abelian groups (#10361) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-meta modifies-tactic-syntax awaiting-author help-wanted 439/0 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/MAbel.lean,MathlibTest/mabel.lean 4 10 ['BoltonBailey', 'dignissimus', 'github-actions', 'joneugster', 'kbuzzard'] joneugster
assignee:joneugster
109-77367
3 months ago
114-58963
3 months ago
0-16
16 seconds
21501 sksgurdldi
author:sksgurdldi
feat(List): add sum_zipWith_eq_finset_sum ### **Description:** This PR adds the lemma `List.sum_zipWith_eq_finset_sum` to `Mathlib.Algebra.BigOperators.Group.Finset.Basic`. #### **Statement:** The sum of the `zipWith` operation on two lists equals the sum of applying the operation to corresponding elements of the two lists, indexed over the minimum of their lengths. #### **Formal Statement:** ```lean lemma sum_zipWith_eq_finset_sum [Inhabited α] [Inhabited β] [AddCommMonoid γ] {op : α → β → γ} (l : List α) (m : List β) : (List.zipWith op l m).sum = ∑ x ∈ (Finset.range (Nat.min l.length m.length)), op (l[x]!) (m[x]!) ``` #### **Remarks:** - This lemma provides a useful equivalence between `List.zipWith` and summation over a `Finset.range` indexed by `Nat.min l.length m.length`. - It can be helpful in algebraic manipulations involving list-based summations. #### **Dependencies:** No additional dependencies. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra awaiting-author
label:t-algebra$
43/0 Mathlib/Algebra/BigOperators/Group/Finset/Basic.lean 1 1 ['github-actions', 'j-loreaux'] nobody
109-76446
3 months ago
109-76446
3 months ago
13-33168
13 days
22302 CharredLee
author:CharredLee
feat: add `CategoryTheory.Topos.Power` This is a continuation of #21281 with the end goal of defining topoi in Mathlib. It introduces the notion of a power object in a category with a subobject classifier, which is a special case of an internal hom. The definition `HasPowerObjects C` contained in this PR is all that remains before `IsTopos C` can be defined. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-category-theory awaiting-author 312/0 Mathlib.lean,Mathlib/CategoryTheory/Topos/Power.lean 2 2 ['github-actions', 'joelriou'] b-mehta
assignee:b-mehta
103-77642
3 months ago
103-78769
3 months ago
0-1528
25 minutes
22390 YunkaiZhang233
author:YunkaiZhang233
feat(CategoryTheory): implemented proofs for factorisation categories being equivalent to iterated comma categories in two ways Completed one of the tasks in TODOs, shown and implemented the details for `(X/C)/f ≌ Factorisation f ≌ f/(C/Y)`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-category-theory awaiting-author 112/1 Mathlib/CategoryTheory/Category/Factorisation.lean 1 9 ['YunkaiZhang233', 'github-actions', 'joelriou'] nobody
98-31875
3 months ago
101-27347
3 months ago
0-6513
1 hour
22159 shetzl
author:shetzl
feat: add definition of pushdown automata Add the definition of pushdown automata and their two acceptance conditions: acceptance based on empty stack and acceptance based on final state. Co-authored-by: Tobias Leichtfried --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-computability new-contributor awaiting-author 70/0 Mathlib.lean,Mathlib/Computability/PDA.lean 2 34 ['YaelDillies', 'github-actions', 'madvorak', 'shetzl'] nobody
84-38789
2 months ago
84-38789
2 months ago
20-81771
20 days
18091 tukamilano
author:tukamilano
feat: Hoeffding's lemma Formalize Hoeffding's lemma using the property of cumulant. Co-authored-by: Yuma Mizuno [mizuno.y.aj@gmail.com](mailto:mizuno.y.aj@gmail.com) --- - [x] depends on: #20151 large-import new-contributor t-measure-probability awaiting-author 339/0 Mathlib.lean,Mathlib/Probability/Hoeffding.lean,Mathlib/Probability/Moments/Basic.lean,Mathlib/Probability/Moments/MGFAnalytic.lean,docs/references.bib 5 55 ['RemyDegenne', 'YaelDillies', 'github-actions', 'mathlib4-dependent-issues-bot', 'tukamilano', 'yuma-mizuno'] tukamilano
assignee:tukamilano
81-30405
2 months ago
81-30413
2 months ago
1-58489
1 day
22355 xyzw12345
author:xyzw12345
feat(Algebra/RingQuot): Some lemmas about `RingQuot.mkAlgHom` and `RingQuot.mkRingHom` This PR provides a few basic lemmas about `RingQuot.mkRingHom` and `RingQuot.mkAlgHom`. These lemmas are about when are two elements mapped to the same one under these two maps, and they correspond to the lemma `Quot.eq`. PR #22279 depends on these lemmas. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra awaiting-author
label:t-algebra$
16/0 Mathlib/Algebra/RingQuot.lean 1 13 ['Paul-Lez', 'erdOne', 'eric-wieser', 'github-actions', 'ocfnash', 'xyzw12345'] nobody
68-52022
2 months ago
69-39345
2 months ago
32-33842
32 days
20671 thefundamentaltheor3m
author:thefundamentaltheor3m
feat(Analysis/Asymptotics/SpecificAsymptotics): Proving that 𝛔ₖ(n) = O(nᵏ⁺¹) This PR proves a result about the $\sigma_k(n)$ arithmetic function, namely, that it is $O\left(n^{k+1}\right)$. Main theorem: `theorem sigma_asymptotic (k : ℕ) : (fun n ↦ (σ k n : ℝ)) =O[atTop] (fun n ↦ (n ^ (k + 1) : ℝ))` This result was proved as part of the sphere packing project. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import new-contributor t-number-theory awaiting-author 29/0 Mathlib/Analysis/Asymptotics/SpecificAsymptotics.lean 1 2 ['b-mehta', 'github-actions'] b-mehta
assignee:b-mehta
63-21305
2 months ago
73-15782
2 months ago
9-59130
9 days
21903 yhtq
author:yhtq
feat: add from/toList between `FreeSemigroup` and `List` with relative theorems Add from/toList between `FreeSemigroup` and `List` with relative theorems, as well as an incidental definition of lexicographic order on `FreeSemigroup`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import new-contributor t-algebra awaiting-CI
label:t-algebra$
169/0 Mathlib/Algebra/Free.lean 1 11 ['YaelDillies', 'github-actions'] nobody
62-54115
2 months ago
62-54115
2 months ago
51-9403
51 days
22657 Xmask19
author:Xmask19
feat: a graph is maximally acyclic iff it is a tree --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-combinatorics 86/0 Mathlib/Combinatorics/SimpleGraph/Acyclic.lean 1 6 ['Rida-Hamadani', 'b-mehta', 'github-actions', 'grunweg'] b-mehta
assignee:b-mehta
62-19772
2 months ago
62-19793
2 months ago
84-10469
84 days
23949 Louddy
author:Louddy
feat: SkewPolynomial # Univariate skew polynomials Skew polynomials are represented as `SkewMonoidAlgebra R (Multiplicative ℕ)`, where `R` is usually at least a Semiring. In this file, we define `SkewPolynomial` and provide basic instances. This is currently missing the definition of `coeff` and `single` as they require a more advance interface of `SkewMonoidAlgebra` which is still WIP (See TODOs in file). Co-authored-by: María Inés de Frutos Fernández <[mariaines.dff@gmail.com](mailto:mariaines.dff@gmail.com)> --- - [ ] depends on: #22078 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import new-contributor t-algebra blocked-by-other-PR
label:t-algebra$
600/42 Mathlib.lean,Mathlib/Algebra/SkewMonoidAlgebra/Basic.lean,Mathlib/Algebra/SkewPolynomial/Basic.lean,docs/references.bib 4 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
59-20722
1 month ago
59-20723
1 month ago
0-2389
39 minutes
23637 kirilvino
author:kirilvino
feat(Combinatorics/SimpleGraph): every circuit contains a cycle proof circuit to cycle proof --- This PR uses the bypass definition in a new function for closed walks that removes repeated vertices. Then proves if the closed walk given is a circuit, that the result from this function is a cycle. This is then packaged up similar to the existing ToPath definition, creating a way of transforming a circuit into a cycle. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-combinatorics awaiting-author 26/0 Mathlib/Combinatorics/SimpleGraph/Path.lean 1 8 ['b-mehta', 'github-actions', 'kirilvino'] nobody
53-37204
1 month ago
53-83825
1 month ago
13-19789
13 days
22925 ggranberry
author:ggranberry
feat(Mathlib/PlaceHolder/ToeplitzHausdorff): Toeplitz-Hausdorff --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-analysis awaiting-author WIP help-wanted 411/0 Mathlib/PlaceHolder/ToeplitzHausdorff.lean,Mathlib/PlaceHolder/ToeplitzHausdorff_v2.lean 2 10 ['faenuccio', 'ggranberry', 'github-actions'] faenuccio
assignee:faenuccio
52-84002
1 month ago
52-84002
1 month ago
4-24257
4 days
23990 robertmaxton42
author:robertmaxton42
feat (Types.Colimits): Quot is functorial and colimitEquivQuot is natural Add `Functor.quotFunctor` to parallel `Functor.sectionsFunctor`, witnessing that `Quot` is functorial; add `colimNatIsoQuotFunctor` to parallel `limNatIsoSectionsFunctor`, witnessing that `colimitEquivQuot` is natural in the diagram $F$. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-category-theory awaiting-author 33/0 Mathlib/CategoryTheory/Limits/Types/Colimits.lean 1 4 ['github-actions', 'joelriou', 'robertmaxton42'] nobody
49-15397
1 month ago
49-15397
1 month ago
8-28043
8 days
22349 dtumad
author:dtumad
feat(Control): Laws for monads with compatible `failure` operation Add a class for a `Monad` that also has an `Alternative` instance, and a class `LawfulAlternative` for types where the failure and monad structures are compatible in the expected way. --- I'm not sure if this should instead go in `Batteries.Control` instead of mathlib, or at least lemmas like `OptionT.run_failure` maybe should. Some of the instances like `Set` would still need to be added in mathlib either way. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-meta WIP 74/3 Mathlib.lean,Mathlib/Control/Lawful.lean,Mathlib/Control/Monad/AlternativeMonad.lean 3 8 ['dtumad', 'eric-wieser', 'github-actions', 'quangvdao'] nobody
44-55296
1 month ago
44-55450
1 month ago
1-20563
1 day
24394 wwylele
author:wwylele
feat(Analysis/Asymptotics): Add filter operation theorems to `IsEquivalent` These are simply restating the corresponding theorems for `isLittleO`, but adding them provides better discovery when one is not familiar with how `IsEquivalent` is defined. I tagged `isEquivalent_map` as `@[simp]` because all of `isBigOWith/isBigO/isLittleO_map` are tagged, but I am not sure if this appropriate. Please let me know if I should remove the tag --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-analysis 13/0 Mathlib/Analysis/Asymptotics/AsymptoticEquivalent.lean 1 1 ['github-actions'] nobody
44-3314
1 month ago
44-3314
1 month ago
44-3373
44 days
22809 b-reinke
author:b-reinke
feat: Category algebras and path algebras This PR defines the category algebra of a linear category and path algebras of quivers. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra t-category-theory WIP
label:t-algebra$
218/0 Mathlib/Algebra/Ring/Assoc.lean,Mathlib/CategoryTheory/Linear/CategoryAlgebra.lean,Mathlib/Combinatorics/Quiver/PathAlgebra.lean,Mathlib/Data/DFinsupp/BigOperators.lean 4 2 ['b-reinke', 'github-actions'] nobody
37-45186
1 month ago
37-45186
1 month ago
0-0
0 seconds
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$
48/24 Mathlib/Topology/Algebra/Module/FiniteDimension.lean,Mathlib/Topology/Algebra/Module/ModuleTopology.lean 2 5 ['erdOne', 'github-actions', 'matthewjasper'] nobody
37-13321
1 month ago
37-30391
1 month ago
38-85090
38 days
15649 TpmKranz
author:TpmKranz
feat(Computability): introduce Generalised NFA as bridge to Regular Expression Lays the groundwork for a proof of equivalence of NFA and RE, w.r.t. described language. Actual connection to NFA comes later, after the groundwork for the opposite direction has been laid. Second chunk of #12648 --- - [x] depends on: #15647 [Data.FinEnum.Option unchanged since then] [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-zulip t-computability new-contributor awaiting-author 298/0 Mathlib.lean,Mathlib/Computability/GNFA.lean,Mathlib/Computability/Language.lean,Mathlib/Computability/RegularExpressions.lean,docs/references.bib 5 6 ['github-actions', 'mathlib4-dependent-issues-bot', 'meithecatte', 'trivial1711'] nobody
34-77905
1 month ago
34-77914
1 month ago
23-54870
23 days
20648 anthonyde
author:anthonyde
feat: formalize regular expression -> εNFA The file `Computability/RegularExpressionsToEpsilonNFA.lean` contains a formal definition of Thompson's method for constructing an `εNFA` from a `RegularExpression` and a proof of its correctness. --- - [x] depends on: #20644 - [x] depends on: #20645 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-zulip t-computability new-contributor 490/0 Mathlib.lean,Mathlib/Computability/RegularExpressionsToEpsilonNFA.lean,docs/references.bib 3 5 ['github-actions', 'mathlib4-dependent-issues-bot', 'meithecatte', 'qawbecrdtey'] nobody
34-77216
1 month ago
34-77851
1 month ago
75-77754
75 days
24361 Hagb
author:Hagb
feat(Data/Finsupp/MonomialOrder): `0 ≤ a` where `a : m.syn` `simp` would be able to solve it. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data new-contributor easy 3/0 Mathlib/Data/Finsupp/MonomialOrder.lean 1 1 ['github-actions'] nobody
33-42488
1 month ago
33-42488
1 month ago
45-44165
45 days
24172 LessnessRandomness
author:LessnessRandomness
feat: specialize rational root theorem to usual rational numbers and integers Rational root theorem and integral root theorem - the special case for usual rational numbers and integers. --- new-contributor t-algebra
label:t-algebra$
123/0 Mathlib.lean,Mathlib/RingTheory/Polynomial/OfRationalNumbers/RationalRootTheorem.lean 2 2 ['github-actions', 'grunweg'] mariainesdff
assignee:mariainesdff
32-46491
1 month ago
52-14174
1 month ago
52-14228
52 days
24637 michaellee94
author:michaellee94
feat(Analysis/ODE/MaximalSolution): Existence of maximal solutions for ODE meeting Picard-Lindelöf conditions Add existence proof for maximal solution of ODE using Picard-Lindelöf and a uniqueness theorem using Grönwall's lemma. --- - [ ] depends on: #20704 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-analysis blocked-by-other-PR 746/1 Mathlib.lean,Mathlib/Analysis/ODE/MaximalSolution.lean,docs/undergrad.yaml 3 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'michaellee94'] nobody
31-70108
1 month ago
32-6233
1 month ago
2-10512
2 days
22314 shetzl
author:shetzl
feat: add leftmost derivations for context-free grammars Leftmost derivations are often easier to reason about than arbitrary derivations. This PR adds leftmost variants of Rewrites, Produces and Derives to the existing definition of context-free grammars and proves that a string of terminals can be derived iff it can be leftmost derived. Co-authored-by: Tobias Leichtfried --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-computability new-contributor awaiting-author 383/0 Mathlib.lean,Mathlib/Computability/LeftmostDerivation.lean 2 54 ['YaelDillies', 'github-actions', 'madvorak', 'shetzl'] YaelDillies
assignee:YaelDillies
31-36180
1 month ago
31-36180
1 month ago
72-3718
72 days
22196 xyzw12345
author:xyzw12345
feat: `lie_ring` tactic and `LieReduce` command In this PR, we implement a new tactic that reduces expressions in a `LieRing` to a normal form and checks whether they are equal, and a command which reduces the expression and displays the normal form. The implementation of this tactic imitates the `ring` tactic, using the `Qq` package to implement a specific reduction algorithm, following the theory of Hall sets and Lyndon words. A reference for the algorithm can be found at, for example, [here](https://personal.math.ubc.ca/~cass/research/pdf/Free.pdf). This project is the result of a workshop at Peking University, and @siddhartha-gadgil has helped us a lot on understanding the concepts in metaprogramming. Edit: The changes are reverted to a point where only `AtomM` is used. Co-authored-by: @Thmoas-Guan <2300010733@stu.pku.edu.cn> @yhtq <2100012990@stu.pku.edu.cn> @Blackfeather007 <2100017455@stu.pku.edu.cn> --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-meta 816/2 Mathlib.lean,Mathlib/Algebra/Lie/Derivation/AdjointAction.lean,Mathlib/Tactic.lean,Mathlib/Tactic/LieAlgebra/Basic.lean,Mathlib/Tactic/LieAlgebra/LieRingNF.lean,Mathlib/Util/AtomM.lean,MathlibTest/lie_ring.lean,scripts/noshake.json 8 16 ['bryangingechen', 'eric-wieser', 'faenuccio', 'github-actions', 'grunweg', 'ocfnash', 'siddhartha-gadgil', 'xyzw12345'] robertylewis
assignee:robertylewis
31-30093
1 month ago
106-61592
3 months ago
106-61583
106 days
24036 Louddy
author:Louddy
feat: add `HeightOneSpectrum.ofPrime` Add a definition relating elements of type `HeightOneSpectrum R` with the (nonzero) prime elements of the monoid with zero `Ideal R`. (Note the distinction between `Prime` and `Ideal.IsPrime`). The documentation string is inspired from [Ideal.prime_iff_isPrime](https://leanprover-community.github.io/mathlib4_docs/Mathlib/RingTheory/DedekindDomain/Ideal.html#Ideal.prime_iff_isPrime). This was discussed [#mathlib4 > Placing a definition in `DedekindDomain.Ideal` @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Placing.20a.20definition.20in.20.60DedekindDomain.2EIdeal.60/near/511647129). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra
label:t-algebra$
11/1 Mathlib/RingTheory/DedekindDomain/Ideal.lean 1 5 ['Louddy', 'Ruben-VandeVelde', 'github-actions'] Ruben-VandeVelde
assignee:Ruben-VandeVelde
31-28220
1 month ago
56-29490
1 month ago
56-29544
56 days
24008 meithecatte
author:meithecatte
chore(EpsilonNFA): replace manual lemmas with @[simps] --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-computability new-contributor awaiting-author 2/24 Mathlib/Computability/EpsilonNFA.lean 1 2 ['YaelDillies', 'github-actions', 'urkud'] nobody
29-37044
29 days ago
29-37044
29 days ago
27-52316
27 days
21985 FernandoChu
author:FernandoChu
feat(CategoryTheory): the Grothendieck construction is prefibered Adds a `isPreFibered` instance for the Grothendieck construction. Co-authored-by: Christian Merten --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-category-theory awaiting-author 55/0 Mathlib/CategoryTheory/Bicategory/Functor/Pseudofunctor.lean,Mathlib/CategoryTheory/Bicategory/Grothendieck.lean 2 15 ['callesonne', 'chrisflav', 'github-actions'] nobody
28-82913
28 days ago
68-14237
2 months ago
8-4256
8 days
22948 pelicanhere
author:pelicanhere
feat(Algebra/DirectSum): morphism of directsum decomposition Define morphism of directsum decomposition, which would be later used in defineing graded ring hom. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra
label:t-algebra$
83/0 Mathlib/Algebra/DirectSum/Decomposition.lean 1 9 ['eric-wieser', 'github-actions', 'pelicanhere'] eric-wieser
assignee:eric-wieser
28-41099
28 days ago
86-37917
2 months ago
86-37959
86 days
24372 Hagb
author:Hagb
feat(Tactic/SimpIntro): add support for introducing non-propositions `simp_intro` would be able to introduce non-propositions. The previous `simp_intro` tactic cannot solve some statement that can be solved by applying `intro` and `simp` like `simp_intro`. For example, the following one can be solved like this ```lean example (r : Nat → Prop) : (∀ x, x > 0 → r x) → ∀ y z, y = 0 → z > y → r z := by simp intro hr try simp at hr -- does nothing try simp [hr] -- does nothing intro y z try simp [hr] -- does nothing intro hy try simp [hr] at hy -- does nothing simp [hr, hy] intro hyz try simp [hr, hy] at hyz simp [hr, hy, hyz] -- accomplish the goal successfully ``` while the previous `simp_intro` cannot introduce `y` and `z` here. ```lean example (r : Nat → Prop) : (∀ x, x > 0 → r x) → ∀ y z, y = 0 → z > y → r z := by /- the previous `simp_intro` fails with message: invalid 'simp', proposition expected Nat -/ simp_intro .. -- or `simp_intro hr y` example (r : Nat → Prop) : (∀ x, x > 0 → r x) → ∀ y z, y = 0 → z > y → r z := by -- unsolved simp_intro hr example (r : Nat → Prop) : (∀ x, x > 0 → r x) → ∀ y z, y = 0 → z > y → r z := by -- successfully solve the goal with the `simp_intro` in thie commit simp_intro .. -- or `simp_intro hr y z hy hz` ``` This commit makes it be able to introduce these kinds of hypotheses. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-meta 13/2 Mathlib/Tactic/SimpIntro.lean,MathlibTest/simp_intro.lean 2 1 ['github-actions'] kmill
assignee:kmill
27-81860
27 days ago
45-5392
1 month ago
45-5443
45 days
24395 rudynicolop
author:rudynicolop
feat(Data/List): list splitting definitions and lemmas Adds definitions and lemmas for obtaining all prefixes and suffixes of lists. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data new-contributor 143/2 Mathlib/Data/List/Perm/Lattice.lean,Mathlib/Data/List/TakeDrop.lean 2 1 ['github-actions'] ericrbg
assignee:ericrbg
27-81842
27 days ago
44-2869
1 month ago
44-2931
44 days
23955 Louddy
author:Louddy
feat: Ideal.count_associates_eq Add variant of `UniqueFactorizationMonoid.count_normalizedFactors_eq` for associated Ideals. This is convenient when you need to talk about an element as `a₀ = x ^ n * a`. Note the file is slightly over the 1500 lines limit, I hope that is ok. 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/) new-contributor t-algebra
label:t-algebra$
35/1 Mathlib/RingTheory/DedekindDomain/Ideal.lean 1 7 ['Louddy', 'Ruben-VandeVelde', 'alreadydone', 'github-actions', 'grunweg'] kbuzzard
assignee:kbuzzard
26-44624
26 days ago
26-44624
26 days ago
53-45384
53 days
18379 oeb25
author:oeb25
feat(Topology/ENNReal): Add `ENNReal.tsum_biUnion` This adds infinite versions of `Finset.sum_biUnion` to `ENNReal`s. --- One notable difference from the `Finset` version is that for `tsum` we have two ways for selecting the summands: `∑' x : ⋃ i ∈ S` or `∑' x : ⋃ i, t i`. This PR adds both. I tried to extend this beyond `ENNReal`, but didn't find a clean way to do it. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-topology 34/0 Mathlib/Data/Set/Lattice.lean,Mathlib/Data/Set/Pairwise/Lattice.lean,Mathlib/Topology/Instances/ENNReal/Lemmas.lean 3 12 ['github-actions', 'grunweg', 'j-loreaux', 'oeb25'] nobody
25-33393
25 days ago
25-34406
25 days ago
127-82912
127 days
22078 Louddy
author:Louddy
feat(SkewMonoidAlgebra): multiplication and algebraic instances # Multiplication and Algebraic Instances In this PR, we introduce the definition of the skewed convolution product on `SkewMonoidAlgebra k G`. Here, the product of two elements `f g : SkewMonoidAlgebra k G` is the finitely supported function whose value at `a` is the sum of `f x * (x • g y)` over all pairs `x, y` such that `x * y = a`. We also introduce the associated algebraic instances. ## Context This is the third part of a planned series of PRs aiming to formalise skew monoid algebras. The PRs are split to ease the review process. The moral sum of these planned PRs is #10541. The first and second part were #15878 and #19084. Co-authored-by: María Inés de Frutos Fernández <[mariaines.dff@gmail.com](mailto:mariaines.dff@gmail.com)> --- [![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$
453/45 Mathlib/Algebra/SkewMonoidAlgebra/Basic.lean 1 57 ['AntoineChambert-Loir', 'Louddy', 'github-actions', 'kbuzzard'] nobody
24-42459
24 days ago
26-39366
26 days ago
98-59896
98 days
5919 MithicSpirit
author:MithicSpirit
feat: implement orthogonality for AffineSubspace Define `AffineSubspace.orthogonal` and `AffineSubspace.IsOrtho`, as well as develop an API emulating that of `Submodule.orthogonal` and `Submodule.IsOrtho`, respectively. Additionally, provide some relevant lemmas exclusive to affine subspaces, which are mostly to do with the relationship between orthogonality and `AffineSubspace.Parallel`. Closes #5539 --- Still WIP as I need to add more docstrings as well as notations for the new definitions. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-analysis WIP help-wanted 287/0 Mathlib.lean,Mathlib/Analysis/InnerProductSpace/AffineSubspace.lean 2 6 ['MithicSpirit', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant'] MithicSpirit
assignee:MithicSpirit
23-7190
23 days ago
23-7208
23 days ago
0-0
0 seconds
22503 Kevew
author:Kevew
chore(Nat): Nat factorization multiplicity Ported lemmas from `Data/Nat/Multiplicity` to into a new file called `Data/Nat/Factorization/Multiplicity`, re-written in terms of `factorization`. --- - [x] depends on: #24576 - [ ] depends on: #25002 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-data new-contributor blocked-by-other-PR 327/101 Mathlib.lean,Mathlib/Data/Nat/Factorization/Basic.lean,Mathlib/Data/Nat/Factorization/LCM.lean,Mathlib/Data/Nat/Factorization/Multiplicity.lean,Mathlib/Data/Nat/Multiplicity.lean,Mathlib/GroupTheory/Exponent.lean,Mathlib/NumberTheory/Cyclotomic/PrimitiveRoots.lean,Mathlib/RingTheory/RootsOfUnity/PrimitiveRoots.lean 8 40 ['Kevew', 'Paul-Lez', 'YaelDillies', 'github-actions', 'grunweg', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] Kevew
assignee:Kevew
22-2003
22 days ago
25-44365
25 days ago
85-42249
85 days
24932 jkanschik
author:jkanschik
feat(Analysis/Calculus/VectorField): Implement product rule for liebrackets This adds lemmas for the product rule (or Leibniz rule) for Lie brackets on vector fields. These new lemmas are called `lieBracket_smul_left` and similar. To accomodate this, rename the existing lemmas `{m}lieBracket{Within}_smul_{left,right}` to `{m}lieBracket{Within}_const_smul_{left,right}`. An additional PR for the same functionality on manifolds is in preparation and would depend on this PR. This will become useful when introducing Lie derivatives or covariant derivatives in differential geometry. new-contributor t-differential-geometry awaiting-author 78/28 Mathlib/Analysis/Calculus/VectorField.lean,Mathlib/Geometry/Manifold/GroupLieAlgebra.lean,Mathlib/Geometry/Manifold/VectorField/LieBracket.lean 3 30 ['github-actions', 'grunweg', 'jkanschik', 'sgouezel'] nobody
22-715
22 days ago
23-30023
23 days ago
1-1522
1 day
24966 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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-differential-geometry 154/13 Mathlib/Geometry/Manifold/PartitionOfUnity.lean 1 3 ['github-actions', 'grunweg', 'michaellee94'] nobody
21-79963
21 days ago
23-17943
23 days ago
23-45496
23 days
19796 peakpoint
author:peakpoint
feat: L'Hopital's rule from within a convex set --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-analysis 190/19 Mathlib/Algebra/Polynomial/Module/Basic.lean,Mathlib/Analysis/Calculus/LHopital.lean,Mathlib/Analysis/Convex/Topology.lean,Mathlib/Geometry/Manifold/Instances/Real.lean,Mathlib/Order/Interval/Set/Basic.lean 5 14 ['RemyDegenne', 'github-actions', 'leanprover-community-bot-assistant', 'peakpoint', 'sgouezel'] sgouezel
assignee:sgouezel
21-79134
21 days ago
21-79134
21 days ago
55-29418
55 days
20913 Thmoas-Guan
author:Thmoas-Guan
feat(Algebra): Define the associated graded ring to filtered ring. Define the associated graded ring to a filtered ring. --- - [x] depends on: #20900 - [x] depends on: #22230 - [ ] depends on: #22631 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra blocked-by-other-PR
label:t-algebra$
442/0 Mathlib.lean,Mathlib/RingTheory/FilteredAlgebra/AssociatedGraded.lean 2 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
20-35139
20 days ago
20-35158
20 days ago
0-70480
19 hours
21806 Thmoas-Guan
author:Thmoas-Guan
feat(Algebra): associated graded algebra Define the associated graded algebra of a filtered algebra, constructed from a special case of associated graded ring. --- - [x] depends on: #20900 - [ ] depends on: #20913 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra blocked-by-other-PR WIP
label:t-algebra$
552/0 Mathlib.lean,Mathlib/RingTheory/FilteredAlgebra/AssociatedGraded.lean 2 n/a ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
20-35082
20 days ago
unknown
unknown
20940 Thmoas-Guan
author:Thmoas-Guan
feat(Algebra): Associated graded module Define the associated graded module to a filtered module. --- - [x] depends on: #20900 - [ ] depends on: #20913 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra blocked-by-other-PR WIP
label:t-algebra$
656/0 Mathlib.lean,Mathlib/RingTheory/FilteredAlgebra/AssociatedGraded.lean 2 n/a ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] Blackfeather007
assignee:Blackfeather007
20-34999
20 days ago
unknown
unknown
22632 Thmoas-Guan
author:Thmoas-Guan
feat(Algebra): define filtered add group hom In this file we define filtered hom and the corresponding associated graded hom for abelian groups. Co-authored-by: Huanyu Zheng @Yu-Misaka Co-authored-by: Yi Yuan @yuanyi-350 Co-authored-by: Weichen Jiao @AlbertJ-314 --- - [ ] depends on: #22631 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra blocked-by-other-PR
label:t-algebra$
378/0 Mathlib.lean,Mathlib/RingTheory/FilteredAlgebra/AssociatedGraded.lean,Mathlib/RingTheory/FilteredAlgebra/FilteredHom.lean 3 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
20-34810
20 days ago
20-34831
20 days ago
0-1204
20 minutes
22208 Thmoas-Guan
author:Thmoas-Guan
feat(Algebra):filtered ring hom In this PR, we define the filtered ring morphisms on rings and prove some basic properties of them. Co-authored-by: Huanyu Zheng @Yu-Misaka Co-authored-by: Yi Yuan @yuanyi-350 Co-authored-by: Weichen Jiao @AlbertJ-314 --- - [ ] depends on: #20913 - [ ] depends on: #22632 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra blocked-by-other-PR
label:t-algebra$
812/0 Mathlib.lean,Mathlib/RingTheory/FilteredAlgebra/AssociatedGraded.lean,Mathlib/RingTheory/FilteredAlgebra/FilteredHom.lean 3 n/a ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
20-34730
20 days ago
unknown
unknown
22707 Thmoas-Guan
author:Thmoas-Guan
feat(Algebra): associated graded exact of exact and strict In this file, we define the concept of exhaustive filtrations. We also prove a AssociatedGradedRingHom sequence is exact iff each GradedPieceHom is exact. And when a sequence is strict exact, the corresponding AssociatedGradedRingHom sequence is also exact. Co-authored-by: Huanyu Zheng @Yu-Misaka Co-authored-by: Yi Yuan @yuanyi-350 Co-authored-by: Weichen Jiao @AlbertJ-314 --- - [ ] depends on: #22632 - [x] depends on: #22705 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra blocked-by-other-PR
label:t-algebra$
534/0 Mathlib.lean,Mathlib/RingTheory/FilteredAlgebra/AssociatedGraded.lean,Mathlib/RingTheory/FilteredAlgebra/Exactness.lean,Mathlib/RingTheory/FilteredAlgebra/FilteredHom.lean 4 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
20-34552
20 days ago
20-34573
20 days ago
0-464
7 minutes
22972 Thmoas-Guan
author:Thmoas-Guan
feat(Algebra): exact of associated graded exact We proved that a chain complex is exact if its associated graded complex is exact. Co-authored-by: Huanyu Zheng @Yu-Misaka Co-authored-by: Yi Yuan @yuanyi-350 Co-authored-by: Weichen Jiao @AlbertJ-314 --- - [ ] depends on: #22632 - [x] depends on: #22705 - [ ] depends on: #22707 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra blocked-by-other-PR
label:t-algebra$
729/0 Mathlib.lean,Mathlib/RingTheory/FilteredAlgebra/AssociatedGraded.lean,Mathlib/RingTheory/FilteredAlgebra/Exactness.lean,Mathlib/RingTheory/FilteredAlgebra/FilteredHom.lean 4 n/a ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
20-34488
20 days ago
unknown
unknown
24206 LessnessRandomness
author:LessnessRandomness
feat(Geometry/Euclidean/Angle/Unoriented): triangle inequality for angles Replace `proof_wanted` with proof. --- new-contributor t-euclidean-geometry awaiting-author 221/11 Mathlib.lean,Mathlib/Geometry/Euclidean/Angle/Unoriented/Affine.lean,Mathlib/Geometry/Euclidean/Angle/Unoriented/Basic.lean,Mathlib/Geometry/Euclidean/Angle/Unoriented/TriangleInequality.lean 4 16 ['LessnessRandomness', 'Timeroot', 'github-actions', 'jsm28', 'urkud'] jsm28
assignee:jsm28
19-77809
19 days ago
30-84002
30 days ago
20-6326
20 days
20240 mitchell-horner
author:mitchell-horner
feat(Combinatorics/SimpleGraph): prove the Kővári–Sós–Turán theorem Prove the Kővári–Sós–Turán theorem for simple graphs: the `(completeBipartiteGraph α β).Free` simple graphs for `card α ≤ card β` on the vertex type `V` have at most `(card β-1)^(1/(card α))*(card V)^(2-1/(card α))/2 + (card V)*(card α-1)/2` edges. --- - [x] depends on: #19865 - [x] depends on: #20738 I'd like to make `aux` not private in the `KovariSosTuran` namespace to enable reuse of the double-counting here, but I don't know what to call it. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-combinatorics 289/0 Mathlib.lean,Mathlib/Combinatorics/SimpleGraph/Bipartite.lean,Mathlib/Combinatorics/SimpleGraph/Extremal/KovariSosTuran.lean 3 3 ['github-actions', 'mathlib4-dependent-issues-bot'] awainverse
assignee:awainverse
19-29414
19 days ago
41-69299
1 month ago
41-69833
41 days
22018 maddycrim
author:maddycrim
feat(RingTheory/Localization/Pi): localization of a finite direct product where each semiring in product has maximal nilradical is a projection For noncomputable def `surjectivePiNilradicalIsMaximal` : Let `M` be a submonoid of a direct product of commutative rings `R i`. If each `R i` has maximal nilradical then the direct product `∏ R i` surjects onto the localization of `∏ R i` at `M`. --- [![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$
28/0 Mathlib/RingTheory/Localization/Pi.lean 1 24 ['Paul-Lez', 'alreadydone', 'erdOne', 'github-actions', 'grunweg', 'jcommelin', 'maddycrim'] mariainesdff
assignee:mariainesdff
19-29279
19 days ago
64-12686
2 months ago
110-85911
110 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
18-68272
18 days ago
46-65829
1 month ago
46-65883
46 days
24139 yuanyi-350
author:yuanyi-350
feat: add `Fin.cycleIcc` which rotates `range(i, j)` In this file, I define permutation `cycleIcc i j hij`, which is the cycle `(i i+1 .... j)` leaving `(0 ... i-1)` and `(j+1 ... n-1)` unchanged. In other words, it rotates elements in `[i, j]` one step to the right. Also I prove some properties of `cycleIcc i j hij` such as it is a cycle and its cycleType is `j - i` **This definition is used to prove the following result:** ``` theorem succAbove_comp_cycleIcc [NeZero n] (x : Fin (n + 1) → L) (i j : Fin (n + 1)) (eq : x i = x j) (lt : i < j) x ∘ i.succAbove = x ∘ j.succAbove ∘ (cycleIcc hij) ``` More clearly, `x ∘ i.succAbove` and `x ∘ j.succAbove` are `Fin n → L` types. For example, when `n = 6, i = 2, j = 5` and `x i = x j` ``` x ∘ i.succAbove = (x 0, x 1, x 3, x 4, x 5, x 6) x ∘ j.succAbove = (x 0, x 1, x 2, x 3, x 4, x 6) ``` We have ``` (x 0, x 1, x 3, x 4, x 5, x 6) --(cycleIcc)--->(x 0, x 1, x 5, x 3, x 4, x 6) = (x 0, x 1, x 2, x 3, x 4, x 6) ``` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra
label:t-algebra$
132/1 Mathlib/Algebra/Group/Fin/Basic.lean,Mathlib/Data/Fin/Basic.lean,Mathlib/Data/Nat/SuccPred.lean,Mathlib/GroupTheory/Perm/Fin.lean 4 27 ['acmepjz', 'faenuccio', 'github-actions', 'grunweg', 'leanprover-bot', 'leanprover-community-bot-assistant', 'mbkybky', 'yuanyi-350'] faenuccio
assignee:faenuccio
18-23587
18 days ago
38-69996
1 month ago
52-84299
52 days
24651 Hagb
author:Hagb
feat(RingTheory/Finiteness/Defs): span of a set is finitely generated iff generated by a finite subset --- - [ ] depends on: #24648 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra
label:t-algebra$
14/0 Mathlib/RingTheory/Finiteness/Defs.lean 1 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
17-38635
17 days ago
17-38654
17 days ago
17-43206
17 days
24816 ciskiko
author:ciskiko
feat(GroupTheory): add Regular Wreath Product feat: add regular wreath product and some results; add iterated wreath product; add the isomorphism of iterated wreath product of Z_p to sylow p subgroup of S_{p^n}. Needs some work simplifying final result. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) maintainer-merge new-contributor t-algebra
label:t-algebra$
285/1 Mathlib.lean,Mathlib/Algebra/Group/End.lean,Mathlib/Combinatorics/Additive/AP/Three/Behrend.lean,Mathlib/Data/Nat/Multiplicity.lean,Mathlib/GroupTheory/RegularWreathProduct.lean,Mathlib/Logic/Equiv/Fin/Basic.lean,Mathlib/SetTheory/Cardinal/Finite.lean 7 102 ['ciskiko', 'github-actions', 'tb65536'] tb65536
assignee:tb65536
15-33430
15 days ago
15-33431
15 days ago
24-38027
24 days
8102 miguelmarco
author:miguelmarco
feat(Tactic): add `unify_denoms` and `collect_signs` tactics This PR adds four new tactics: - `unify_denoms` tries to put expressions with several divisions in a form with only one division. In the case of fields, it works similarly to `field_simp`, but if the hypothesis about denominators being nonzero are not present, it assumes them, and leaves them as new goals to prove. In that sense, it is an "unsafe" tactic (but can be useful nevertheless, for example when you can't find which exact hypothesis is missing). It also works with expressions of naturals and Euclidean domains, assuming the corresponding hypothesis about the denominators dividing the numerators. - `unify_denoms!` extends `unify_denoms` to work with (in)equalities, assuming also that the denominators, once in normal form, are positive. - `collect_signs` works similarly with expressions using sums and substractions: it tries to put them in a form of one sum minus other sum. In the case of working with naturals, it assumes that we never substract a bigger number from a smaller one. Both are implemented essentially as a macro that combines several rewriting rules. Some new lemmas with the corresponding rules are added. --- new-contributor t-meta please-adopt modifies-tactic-syntax good first issue 407/0 Mathlib.lean,Mathlib/Algebra/EuclideanDomain/Basic.lean,Mathlib/Tactic.lean,Mathlib/Tactic/CollectSigns.lean,Mathlib/Tactic/UnifyDenoms.lean,MathlibTest/unify_denoms.lean,scripts/noshake.json 7 54 ['Paul-Lez', 'YaelDillies', 'github-actions', 'joneugster', 'kbuzzard', 'miguelmarco'] Paul-Lez
assignee:Paul-Lez
14-24186
14 days ago
26-4939
26 days ago
22-16933
22 days
25224 xcloudyunx
author:xcloudyunx
feat(Combinatorics/SimpleGraph): edgeSet of Eulerian walk equal to edgeSet of graph --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-combinatorics easy 6/0 Mathlib/Combinatorics/SimpleGraph/Trails.lean 1 2 ['IvanRenison', 'github-actions'] nobody
12-83709
12 days ago
13-74712
13 days ago
13-75614
13 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'] nobody
12-83102
12 days ago
13-74514
13 days ago
13-74571
13 days
25248 xcloudyunx
author:xcloudyunx
feat(Combinatorics/SimpleGraph): Add Subgraph.inclusion_edge_apply_coe and inclusion_edgeSet_apply_coe --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-combinatorics 12/0 Mathlib/Combinatorics/SimpleGraph/Subgraph.lean 1 1 ['github-actions'] nobody
12-76744
12 days ago
12-76745
12 days ago
12-76800
12 days
25238 Hagb
author:Hagb
feat(Tactic/ComputeDegree): add support for scalar multiplication with different types It would be able to deal with `a • (X : R[X])` where `a : S` is in a different type `S` with `[SMulZeroClass S R]`. --- - [x] depends on: #25237 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor 17/5 Mathlib/Tactic/ComputeDegree.lean,MathlibTest/ComputeDegree.lean 2 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
12-56734
12 days ago
12-81177
12 days ago
12-83080
12 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
12-42970
12 days ago
13-18912
13 days ago
19-23308
19 days
25257 Hagb
author:Hagb
feat(Mathlib/Algebra/Polynomial/Degree/Domain.lean): generalize `natDegree_smul` from `SMulWithZero` to `SMulZeroClass` as suggested by @eric-wieser in https://github.com/leanprover-community/mathlib4/pull/25237#discussion_r2111599865 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra
label:t-algebra$
4/3 Mathlib/Algebra/Polynomial/Degree/Domain.lean 1 1 ['github-actions'] nobody
12-26109
12 days ago
12-26109
12 days ago
12-26171
12 days
25283 Brian-Nugent
author:Brian-Nugent
feat: regular local rings Adds regular local rings and proves they are integral domains. --- - [ ] depends on: #25280 - [ ] depends on: #25282 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra blocked-by-other-PR
label:t-algebra$
871/0 .vscode/settings.json,Mathlib.lean,Mathlib/RingTheory/EmbeddingDimension.lean,Mathlib/RingTheory/LocalRingDimension.lean,Mathlib/RingTheory/RegularLocalRing.lean 5 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
11-84684
11 days ago
11-84686
11 days ago
0-882
14 minutes
25282 Brian-Nugent
author:Brian-Nugent
feat: krull dimension facts for Noetherian local rings Proves that when modding out by a non-unit, the Krull dimension of a noetherian local ring drops by at most one. Also proves that the embedding dimension is an upper bound on the Krull dimension. --- - [ ] depends on: #25280 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra blocked-by-other-PR
label:t-algebra$
626/0 .vscode/settings.json,Mathlib.lean,Mathlib/RingTheory/EmbeddingDimension.lean,Mathlib/RingTheory/LocalRingDimension.lean 4 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
11-84683
11 days ago
11-84685
11 days ago
0-1566
26 minutes
24543 pfaffelh
author:pfaffelh
feat (Topology/Compactness/CompactSystem): Set system of finite unions of sets in a compact system is again a compact system feat (Topology/Compactness/CompactSystem): The set system of finite unions of sets in a compact system is a compact system A compact system is a set system with the following property: If all finite intersections of a sequence in the set system is non-empty, the countable intersection is not empty. Starting with a compact system, consider the finite unions of sets in the copact system. Such sets again form a compact system (`IsCompactSystem.union.isCompactSystem`). --- - [x] depends on: #24541 - [x] depends on: #24542 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-topology blocked-by-other-PR 431/2 Mathlib/Topology/Compactness/CompactSystem.lean 1 4 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
7-82487
7 days ago
7-82487
7 days ago
0-1830
30 minutes
23500 DrLSimon
author:DrLSimon
feat(MeasureTheory/Decomposition): link the clipped sub of positive measures to Jordan decomposition This introduces a new file `Mathlib/MeasureTheory/Decomposition/JordanSub.lean` which develops the Jordan decomposition of the signed measure `μ.toSignedMeasure - ν.toSignedMeasure` for finite measures `μ` and `ν`, expressing it as the pair `(μ - ν, ν - μ)` of mutually singular finite measures. The key tool is the Hahn decomposition theorem, which yields a measurable partition of the space where `μ ≥ ν` and `ν ≥ μ`. Some basic results of `VectorMeasure` are also provided such as `restrict_neg`, `restrict_sub` `restrict_add_restrict_compl` and `Measure.toSignedMeasure_le_iff` within the `JordanSub.lean` file. They could be moved to another more central place (I guess `VectorMeasure/Basic.lean`). Similarly, `Measure.sub_zero` could go to `Sub.lean`. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-measure-probability 209/2 Mathlib.lean,Mathlib/MeasureTheory/Measure/Decomposition/Hahn.lean,Mathlib/MeasureTheory/Measure/Sub.lean,Mathlib/MeasureTheory/VectorMeasure/Basic.lean,Mathlib/MeasureTheory/VectorMeasure/Decomposition/JordanSub.lean 5 132 ['DavidLedvinka', 'DrLSimon', 'EtienneC30', 'github-actions', 'grunweg', 'urkud'] EtienneC30
assignee:EtienneC30
7-44161
7 days ago
7-44161
7 days ago
29-62586
29 days
22069 Raph-DG
author:Raph-DG
feat(LinearMap): Added lemmas relating kernels of linear maps to Submodule.map Added the lemma ne_map_or_ne_kernel_inter_of_lt stating that if A < B as submodules, then for any linear map f, `ker f ⊓ A ≠ ker f ⊓ B ∨ Submodule.map f A ≠ Submodule.map f B`. We also prove the corollaries ker_inter_mono_of_map_eq and map_mono_of_ker_inter_eq. Co-authored-by: Raphael Douglas Giles (raphaeldouglasgiles@gmail.com) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra
label:t-algebra$
30/0 Mathlib/LinearAlgebra/Span/Basic.lean 1 21 ['Paul-Lez', 'Raph-DG', 'github-actions', 'j-loreaux', 'mattrobball'] mattrobball
assignee:mattrobball
7-31078
7 days ago
7-31078
7 days ago
109-70769
109 days
11021 jstoobysmith
author:jstoobysmith
feat(AlgebraicTopology) : add join of augmented SSets This pull-request adds the definition of the join of augmented SSets defined as contravariant functors from `WithInitial SimplexCategory` to `Type u`. In addition it shows that the join of two standard augmented SSets is again an augmented SSets. From this the definition of the join of simplicial sets should follow easily. To aid the above theory, an api for `WithInitial SimplexCategory` has been created, with the notion of the `join` and `split` (forming a sort of inverse to join) of objects in this category are defined. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-category-theory merge-conflict WIP 2137/1 .gitignore,Mathlib.lean,Mathlib/AlgebraicTopology/Join.lean,Mathlib/AlgebraicTopology/SimplexCategory.lean,Mathlib/AlgebraicTopology/SimplexCategoryWithInitial.lean,Mathlib/AlgebraicTopology/SimplicialSet.lean 6 47 ['github-actions', 'jcommelin'] nobody
313-42768
10 months ago
369-37814
1 year ago
1-20125
1 day
12751 Command-Master
author:Command-Master
feat: add lemmas for Nat/Bits, Nat/Bitwise and Nat/Size Remove `@[simp]` from `Nat.bit_false` and `Nat.bit_true`, as `bit0` and `bit1` are deprecated, and add some lemmas to `Bits`, `Bitwise` and `Size`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data new-contributor merge-conflict 66/7 Mathlib/Data/Nat/Bits.lean,Mathlib/Data/Nat/Bitwise.lean,Mathlib/Data/Nat/Multiplicity.lean,Mathlib/Data/Nat/Size.lean 4 26 ['Command-Master', 'Rida-Hamadani', 'Ruben-VandeVelde', 'YaelDillies', 'github-actions', 'jcommelin'] nobody
294-20067
9 months ago
299-36309
9 months ago
54-52408
54 days
9935 jstoobysmith
author:jstoobysmith
feat(AlgebraicTopology): add constructors for horns Added a function that given a simplicial set S and a set of n-1 simplexes satisfying certain conditions, creates a morphism in SSet from a n horn to a simplicial set S. Included also are a series of lemmas and definitions used in this construction. In particular I define a function that takes a m-simplex in a horn, and returns the smallest 'index' of face it factors through, and give a series of lemmas related to this. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra t-topology merge-conflict awaiting-author
label:t-algebra$
462/2 Mathlib/AlgebraicTopology/SimplicialSet.lean 1 15 ['YaelDillies', 'jcommelin', 'jstoobysmith', 'kim-em', 'linesthatinterlace'] nobody
294-19901
9 months ago
325-21226
10 months ago
14-58814
14 days
10006 jstoobysmith
author:jstoobysmith
feat(AlgebraicTopology): homotopy in quasicategories Defined a homotopy between two 1-simplicies in a quasicategories, and proved the property of being homotopic forms an equivalence relation. --- - [ ] depends on: #9935 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-category-theory merge-conflict awaiting-author blocked-by-other-PR 898/1 Mathlib.lean,Mathlib/AlgebraicTopology/Homotopy.lean,Mathlib/AlgebraicTopology/SimplexCategory.lean,Mathlib/AlgebraicTopology/SimplicialSet.lean 4 3 ['joelriou', 'leanprover-community-mathlib4-bot'] nobody
258-45486
8 months ago
258-45486
8 months ago
0-0
0 seconds
14242 js2357
author:js2357
feat: Prove equivalence of `isDedekindDomain` and `isDedekindDomainDvr` Prove that `isDedekindDomainDvr` is equivalent to both `isDedekindDomain` and `isDedekindDomainInv`. Specifically, prove `isDedekindDomainDvr A → isDedekindDomainInv A`, because `isDedekindDomain A → isDedekindDomainDvr A` and `IsDedekindDomain A ↔ IsDedekindDomainInv A` are already in Mathlib. - [x] depends on: #14099 - [x] depends on: #14216 - [ ] depends on: #14237 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra merge-conflict blocked-by-other-PR
label:t-algebra$
269/1 Mathlib.lean,Mathlib/RingTheory/DedekindDomain/Dvr.lean,Mathlib/RingTheory/FractionalIdeal/LocalizedAtPrime.lean,Mathlib/RingTheory/Localization/Basic.lean 4 2 ['github-actions', 'leanprover-community-mathlib4-bot'] nobody
258-5961
8 months ago
258-5961
8 months ago
0-0
0 seconds
16888 metinersin
author:metinersin
feat(ModelTheory/Complexity): Define conjunctive and disjunctive normal forms Define `FirstOrder.Language.BoundedFormula.IsDNF` and `FirstOrder.Language.BoundedFormula.IsCNF`. --- - [ ] depends on: #16887 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-logic merge-conflict blocked-by-other-PR 415/7 Mathlib/ModelTheory/Complexity.lean,Mathlib/ModelTheory/Equivalence.lean,Mathlib/ModelTheory/Syntax.lean 3 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
250-1939
8 months ago
250-1939
8 months ago
0-1045
17 minutes
16887 metinersin
author:metinersin
feat(ModelTheory/Complexity): define conjunctive and disjunctive formulas Defines `FirstOrder.Language.BoundedFormula.IsConjunctive` and `FirstOrder.Language.BoundedFormula.IsDisjunctive`. --- - [ ] depends on: #16885 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-logic merge-conflict blocked-by-other-PR 300/7 Mathlib/ModelTheory/Complexity.lean,Mathlib/ModelTheory/Equivalence.lean,Mathlib/ModelTheory/Syntax.lean 3 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
250-1939
8 months ago
250-1940
8 months ago
0-1299
21 minutes
16889 metinersin
author:metinersin
feat(ModelTheory/Complexity): Normal forms Defines `FirstOrder.Language.BoundedFormula.toDNF` and `FirstOrder.Language.BoundedFormula.toCNF` - given a quantifier-free formula, these construct a semantically equivalent formula in disjunctive normal form and conjunctive normal form, respectively. --- - [ ] depends on: #16888 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-logic merge-conflict blocked-by-other-PR 525/7 Mathlib/ModelTheory/Complexity.lean,Mathlib/ModelTheory/Equivalence.lean,Mathlib/ModelTheory/Syntax.lean 3 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
250-1938
8 months ago
250-1938
8 months ago
0-613
10 minutes
10190 jstoobysmith
author:jstoobysmith
feat(AlgebraicTopology): add Augmented Simplex Category - Added the definition of the category FinLinOrd of finite linear ordered sets. - Added the definition of the augmented simplex category `AugmentedSimplexCategory`, and showed it is the Skeleton of FinLinOrd. - Showed that the category of augmented simplicial objects defined as a comma category is equivalent to the category of functors from `AugmentedSimplexCategory^\op` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra t-topology t-category-theory merge-conflict WIP
label:t-algebra$
720/0 Mathlib.lean,Mathlib/AlgebraicTopology/AugmentedSimplexCategory.lean,Mathlib/AlgebraicTopology/SimplicialObject.lean,Mathlib/Order/Category/FinLinOrd.lean 4 5 ['TwoFX', 'YaelDillies', 'joelriou', 'jstoobysmith'] nobody
243-12137
8 months ago
243-12137
8 months ago
7-63215
7 days
12750 Command-Master
author:Command-Master
feat: define Gray code --- Define binary reflected gray code, both as a permutation of `Nat` and as a permutation of `BitVec n`, and prove some theorems about them. Additionally, remove `@[simp]` from `Nat.bit_false` and `Nat.bit_true`, as `bit0` and `bit1` are deprecated, and add some lemmas to `Bits`, `Bitwise` and `Size`. - [ ] depends on: #12751 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data new-contributor merge-conflict awaiting-author blocked-by-other-PR 226/0 Mathlib.lean,Mathlib/Data/Nat/Bits.lean,Mathlib/Data/Nat/Bitwise.lean,Mathlib/Data/Nat/GrayCode.lean,Mathlib/Data/Nat/Size.lean 5 5 ['Rida-Hamadani', 'alreadydone', 'github-actions', 'grunweg', 'leanprover-community-mathlib4-bot'] nobody
232-24596
7 months ago
232-24596
7 months ago
6-8380
6 days
9605 davikrehalt
author:davikrehalt
feat(Data/Finset & List): Add Lemmas for Sorting and Filtering This PR includes several useful lemmas to the Data/Finset and Data/List modules in Lean's mathlib: 1. `toFinset_filter` (List): Shows that filtering commutes with toFinset. 2. `toFinset_is_singleton_implies_replicate` (List): Shows a list with a singleton toFinset is a List.replicate. 3. `filter_sort_commute` (Finset): Sorting and filtering can be interchanged in Finsets. 4. `Sorted.filter` (List): A sorted list stays sorted after filtering. 5. `Sorted.append_largest` (List): Appending the largest element keeps a list sorted. 6. `sort_monotone_map` (Finset): Relates sorting of a Finset after mapping to sorting of a list. 7. `sort_insert_largest` (Finset): Sorting a Finset with an inserted largest element. 8. `sort_range` (Finset): Sorting a range in a Finset equals the corresponding range list. 9. ~~`filter_eval_true` (List): Filtering a list with a predicate always true keeps the list unchanged.~~ 10. ~~`filter_eval_false` (List): Filtering with an always-false predicate gives an empty list.~~ 11. ~~`pairwise_concat` (List): Iff condition for Pairwise relation in concatenated lists (similar to pairwise_join).~~ 12. `list_map_toFinset` (Finset): toFinset commutes with map under injection --- - [x] depends on: #15952 This is my first PR to mathlib, so I'm not too familiar with etiquette's and more specifically there are two proofs in the PR which uses aesop, and I am not sure if it's frowned upon. I kept the aesop in there for now as I couldn't construct very short proofs otherwise. The sort_range function proof was suggested in https://leanprover.zulipchat.com/#narrow/stream/113489-new-members/topic/Computing.20Finset.20sort.20of.20Finset.20range/near/410346731 by Ruben Van de Velde. Thanks for your time for improving this PR. t-data new-contributor merge-conflict please-adopt awaiting-author 71/0 Mathlib/Data/Finset/Basic.lean,Mathlib/Data/Finset/Image.lean,Mathlib/Data/Finset/Sort.lean,Mathlib/Data/List/Sort.lean 4 30 ['YaelDillies', 'davikrehalt', 'eric-wieser', 'github-actions', 'jcommelin', 'leanprover-community-mathlib4-bot', 'urkud', 'vihdzp'] YaelDillies
assignee:YaelDillies
221-82306
7 months ago
248-51097
8 months ago
12-48560
12 days
14598 Command-Master
author:Command-Master
chore: add typeclasses to unify various `add_top`, `add_eq_top`, etc. Add the four typeclasses `IsTopAbsorbing`, `IsBotAbsorbing`, `NoTopSum`, `NoBotSum`, as additive equivalents for `MulZeroClass` and `NoZeroDivisors`. Add instances of these for `ENNReal`, `WithTop α`, `WithBot α`, `PUnit`, `EReal`, `PartENat`, `Measure`, `Interval` and `Filter`. Also split `Algebra/Order/AddGroupWithTop` to `Algebra/Order/Group/WithTop` and `Algebra/Order/Monoid/WithTop` --- Previous usages of lemmas with quantified names like `WithTop.add_top` have to be changed to just `add_top`. `add_lt_top` is `@[simp]`, in accordance with `ENNReal.add_lt_top` being `@[simp]`. This affects `WithTop.add_lt_top` which previously hadn't been `@[simp]`. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-order t-algebra merge-conflict
label:t-algebra$
264/195 Archive/Wiedijk100Theorems/BallotProblem.lean,Mathlib.lean,Mathlib/Algebra/Order/Group/WithTop.lean,Mathlib/Algebra/Order/GroupWithZero/Canonical.lean,Mathlib/Algebra/Order/Interval/Basic.lean,Mathlib/Algebra/Order/Monoid/Unbundled/Basic.lean,Mathlib/Algebra/Order/Monoid/Unbundled/Defs.lean,Mathlib/Algebra/Order/Monoid/Unbundled/WithTop.lean,Mathlib/Algebra/Order/Monoid/WithTop.lean,Mathlib/Algebra/PUnitInstances/Order.lean,Mathlib/Algebra/Polynomial/Degree/Definitions.lean,Mathlib/Algebra/Polynomial/Monic.lean,Mathlib/Algebra/Tropical/Basic.lean,Mathlib/Analysis/Analytic/Meromorphic.lean,Mathlib/Analysis/Normed/Lp/ProdLp.lean,Mathlib/Analysis/NormedSpace/ENorm.lean,Mathlib/Analysis/SpecialFunctions/JapaneseBracket.lean,Mathlib/Analysis/SpecialFunctions/Log/ENNRealLog.lean,Mathlib/Data/ENNReal/Operations.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/Data/Nat/PartENat.lean,Mathlib/Data/Nat/WithBot.lean,Mathlib/Data/Real/EReal.lean,Mathlib/LinearAlgebra/Lagrange.lean,Mathlib/MeasureTheory/Covering/Differentiation.lean,Mathlib/MeasureTheory/Decomposition/Lebesgue.lean,Mathlib/MeasureTheory/Function/ConditionalExpectation/CondexpL1.lean,Mathlib/MeasureTheory/Function/Jacobian.lean,Mathlib/MeasureTheory/Function/L1Space.lean,Mathlib/MeasureTheory/Function/L2Space.lean,Mathlib/MeasureTheory/Function/LpSeminorm/Basic.lean,Mathlib/MeasureTheory/Function/LpSeminorm/TriangleInequality.lean,Mathlib/MeasureTheory/Function/LpSpace.lean,Mathlib/MeasureTheory/Function/StronglyMeasurable/Basic.lean,Mathlib/MeasureTheory/Function/UniformIntegrable.lean,Mathlib/MeasureTheory/Integral/Bochner.lean,Mathlib/MeasureTheory/Integral/MeanInequalities.lean,Mathlib/MeasureTheory/Integral/SetIntegral.lean,Mathlib/MeasureTheory/Integral/VitaliCaratheodory.lean,Mathlib/MeasureTheory/Measure/Hausdorff.lean,Mathlib/MeasureTheory/Measure/Lebesgue/Basic.lean,Mathlib/MeasureTheory/Measure/LevyProkhorovMetric.lean,Mathlib/MeasureTheory/Measure/MeasureSpace.lean,Mathlib/MeasureTheory/Measure/MeasureSpaceDef.lean,Mathlib/MeasureTheory/Measure/Regular.lean,Mathlib/MeasureTheory/Measure/Typeclasses.lean,Mathlib/NumberTheory/Padics/PadicNumbers.lean,Mathlib/Order/Filter/Pointwise.lean,Mathlib/Probability/Kernel/Defs.lean,Mathlib/Probability/Martingale/Convergence.lean,Mathlib/RingTheory/Multiplicity.lean,Mathlib/RingTheory/MvPowerSeries/NoZeroDivisors.lean,Mathlib/RingTheory/UniqueFactorizationDomain.lean,Mathlib/Topology/EMetricSpace/Defs.lean,Mathlib/Topology/MetricSpace/Bounded.lean,Mathlib/Topology/MetricSpace/HausdorffDistance.lean,Mathlib/Topology/MetricSpace/Lipschitz.lean 57 30 ['Command-Master', 'YaelDillies', 'github-actions'] nobody
215-52872
7 months ago
215-52872
7 months ago
7-45599
7 days
16885 metinersin
author:metinersin
feat(ModelTheory/Complexity): define literals Defines `FirstOrder.Language.BoundedFormula.IsLiteral` and `FirstOrder.Language.BoundedFormula.simpleNot` - an auxiliary operation that takes the negation of a formula and does some simplification. --- - [x] depends on: #16800 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-logic merge-conflict awaiting-author 148/5 Mathlib/ModelTheory/Complexity.lean,Mathlib/ModelTheory/Equivalence.lean,Mathlib/ModelTheory/Semantics.lean,Mathlib/ModelTheory/Syntax.lean 4 20 ['YaelDillies', 'awainverse', 'github-actions', 'mathlib4-dependent-issues-bot', 'metinersin'] nobody
213-8993
7 months ago
213-8993
7 months ago
0-19926
5 hours
13248 hcWang942
author:hcWang942
feat: basic concepts of auction theory ## Description Formalise some core concepts and results in auction theory: this includes definitions for first-price and second-price auctions, as well as several fundamental results and helping lemmas. This is the very first PR of the project formalizing core concepts and results in auction theory. Our group is working on more contributions on the formalization of game theory prefix. Co-authored-by: Ma Jiajun ## Reference Roughgarden, Tim. ***Twenty Lectures on Algorithmic Game Theory***. Cambridge University Press, 2020. [Link](https://www.cambridge.org/core/books/twenty-lectures-on-algorithmic-game-theory/A9D9427C8F43E7DAEF8C702755B6D72B) --- - [x] Will depend on #14163 once that PR is merged. The Fintype lemmas introduced by this PR have been added in that PR and will be removed from here once that PR gets merged ## Current plan for formalization of Game Theory The current plan for the formalizing of Game Theory include: #### 1. Auction Theory. 🎉 _(200+ lines, this PR)_ - Essential definitions of Sealed-bid auction, First-price auction and Second-price auction. - First-price auction has no dominant strategy. - Second-price auction has dominant strategy. (Second-price auction is DSIC) #### 2. Mechanism design & Myerson's Lemma. 🎉 (400+ lines, pending for modification to Mathlib Standard) - Mechanism design An allocation rule is implementable if there exists - Dominant Strategy Incentive Compatible (DSIC) payment rule - An allocation rule is monotone if for every bidder’s gain is nondecreasing w.r.t. her/his bid - Myerson's Lemma Implementable ⇔ Monotone In the above case, the DSIC payment rule is unique. #### 3. von Neumann‘s Minimax Theorem. 🎉 (800+ lines, pending for modification to Mathlib Standard) - Equilibrium in zero sum game - Formalization strategy: via Loomis’s theorem. #### 4. Nash Equilibrium. 🎉 (pending for modification to Mathlib Standard) #### 5. Brouwer fixed-point theorem. (Work in Progress) #### 6. More Mechanism design. (Planning) new-contributor t-logic merge-conflict awaiting-author 204/0 Mathlib.lean,Mathlib/GameTheory/Auction/Basic.lean,docs/references.bib 3 148 ['Shreyas4991', 'YaelDillies', 'eric-wieser', 'faenuccio', 'github-actions', 'grunweg', 'hcWang942', 'tb65536', 'urkud', 'vihdzp'] hcWang942
assignee:hcWang942
208-47825
6 months ago
unknown
unknown
16116 jjdishere
author:jjdishere
feat(Field): add theorems in Stacks Project Chapter 09FA Fields Add theorems in Stacks Project Chapter 09FA Fields that are not in mathlib. Co-authored-by: --- - [x] depends on: #16105 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra merge-conflict WIP
label:t-algebra$
6/2 Mathlib/Algebra/Field/Defs.lean,Mathlib/Algebra/Field/Subfield.lean 2 6 ['github-actions', 'mathlib4-dependent-issues-bot', 'mergify'] nobody
207-9419
6 months ago
208-78227
6 months ago
0-0
0 seconds
16743 agjftucker
author:agjftucker
feat(Analysis/Calculus/Implicit): define HasStrictDerivAt.implicitFunOfBivariate In [this](https://leanprover.zulipchat.com/#narrow/stream/116395-maths/topic/Implicit.20function.20theorem.20in.20familiar.20form) Zulip thread @Komyyy proved the "familiar" implicit function theorem. Then I wrote a proposal for a Mathlib PR. (Updated) it went: 1. `noncomputable def implicitFunOfBivariate {f : X × Y → Z} {p₀ : X × Y} {fx : X →L[𝕜] Z} {fy : Y ≃L[𝕜] Z} (hf₀ : HasStrictFDerivAt f (fx.coprod fy) p₀) : X → Y := ...` 2. `noncomputable def implicitFunOfBivariate' {f : X → Y → Z} {x₀ : X} {y₀ : Y} {fx : X →L[𝕜] Z} {fy : Y ≃L[𝕜] Z} (hfx : ContDiffAt 𝕜 1 (f · y₀) x₀) (hfy : ContDiffAt 𝕜 1 (f x₀ ·) y₀) (hfx₀ : fderiv 𝕜 (f · y₀) x₀ = fx) (hfy₀ : fderiv 𝕜 (f x₀ ·) y₀ = fy) : X → Y := ...` 3. `theorem image_eq_iff_implicitFunOfBivariate {f : X × Y → Z} {p₀ : X × Y} {fx : X →L[𝕜] Z} {fy : Y ≃L[𝕜] Z} (hf₀ : HasStrictFDerivAt f (fx.coprod fy) p₀) : ∀ᶠ p in 𝓝 p₀, f p = f p₀ ↔ hf₀.implicitFunOfBivariate p.1 = p.2 := ...` 4. `theorem implicitFunOfBivariate_hasStrictFDerivAt {f : X × Y → Z} {x₀ : X} {y₀ : Y} {fx : X →L[𝕜] Z} {fy : Y ≃L[𝕜] Z} (hf₀ : HasStrictFDerivAt f (fx.coprod fy) (x₀, y₀)) : HasStrictFDerivAt hf₀.implicitFunOfBivariate (-fy.symm ∘L fx) x₀ := ...` 5. something on the second derivative (or higher). Although my proposal elicited no response, I am making this micro-PR to address points 1, 3 and 4 since some limited enthusiasm had been shown earlier in that thread (admittedly for another proposal made by another person). I am testing the waters; if this PR gets anywhere I may continue to work on points 2 and 5. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-analysis merge-conflict awaiting-author 132/8 Mathlib/Analysis/Calculus/Implicit.lean,Mathlib/LinearAlgebra/BilinearForm/Orthogonal.lean,Mathlib/LinearAlgebra/Span.lean,Mathlib/Order/Filter/Prod.lean 4 4 ['github-actions', 'sgouezel'] sgouezel
assignee:sgouezel
196-38467
6 months ago
196-38467
6 months ago
63-71154
63 days
18646 jxjwan
author:jxjwan
feat(RingTheory): isotypic components --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra merge-conflict
label:t-algebra$
308/0 Mathlib/Order/CompactlyGenerated/Basic.lean,Mathlib/RingTheory/Isotypic.lean,Mathlib/RingTheory/SimpleModule.lean 3 1 ['github-actions'] nobody
196-30997
6 months ago
196-30997
6 months ago
20-16585
20 days
19526 metakunt
author:metakunt
feat:closure properties of numbers that are introspective to polynomials Prove Part 1 of Claim 1.(i) of Theorem 6.1 in https://www3.nd.edu/~andyp/notes/AKS.pdf. ---- Zulip discussion: https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Aks.20primality.20Theorem.206.2E1.20Claim.20.28i.29.20proven new-contributor t-number-theory merge-conflict awaiting-author 57/0 Mathlib.lean,Mathlib/NumberTheory/AKSPrimality.lean 2 10 ['Ruben-VandeVelde', 'github-actions', 'jcommelin', 'kim-em', 'metakunt'] nobody
190-32330
6 months ago
190-32330
6 months ago
0-16072
4 hours
19125 yhtq
author:yhtq
feat: add theorems to transfer `IsGalois` between pairs of fraction rings feat: add theorems to transfer `IsGalois` between pairs of fraction rings. - [x] depends on: #18404 - [x] depends on: #19124 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra merge-conflict
label:t-algebra$
121/0 Mathlib.lean,Mathlib/FieldTheory/Galois/IsFractionRing.lean,Mathlib/RingTheory/Localization/FractionRing.lean 3 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'tb65536'] nobody
178-70242
5 months ago
185-19265
6 months ago
0-4534
1 hour
11156 smorel394
author:smorel394
feat(LinearAlgebra/{TensorProductBasis,Dual}): basis and dual of `PiTensorProduct` Construct a basis of a `PiTensorProduct` of modules given bases of the modules, and relationship between the dual of a `PiTensorProduct` and the `PiTensorProduct` of the duals. Main results: * `Basis.piTensorProduct` (in `LinearAlgebra/TensorProductBasis.lean`): Let `ι` be a `Fintype` and `M` be a family of modules indexed by `ι`. If `b i : κ i → M i` is a basis for every `i` in `ι`, then `fun (p : Π i, κ i) ↦ ⨂ₜ[R] i, b i (p i)` is a basis of `⨂[R] i, M i`. * `PiTensorProduct.dualDistrib` (in `LinearAlgebra/Dual.lean`): The canonical linear map from `⨂[R] i, Dual R (M i)` to `Dual R (⨂[R] i, M i)`, sending `⨂ₜ[R] i, f i` to the composition of `PiTensorProduct.map f` with the linear equivalence `⨂[R] i, R →ₗ R` given by multiplication. * `PiTensorProduct.dualDistribEquiv` (also in `LinearAlgebra/Dual.lean`): A linear equivalence between `⨂[R] i, Dual R (M i)` and `Dual R (⨂[R] i, M i)` when all `M i` are finite free modules. If `f : (i : ι) → Dual R (M i)`, then this equivalence sends `⨂ₜ[R] i, f i` to the composition of `PiTensorProduct.map f` with the natural isomorphism `⨂[R] i, R ≃ R` given by multiplication. - [ ] depends on: #11155 (currently used as the base branch; do not merge without switching it back to `master`!) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import new-contributor t-algebra merge-conflict please-adopt blocked-by-other-PR
label:t-algebra$
166/2 Mathlib/LinearAlgebra/DirectSum/Finsupp.lean,Mathlib/LinearAlgebra/Dual.lean,Mathlib/LinearAlgebra/TensorProduct/Basis.lean 3 4 ['eric-wieser', 'github-actions', 'leanprover-community-mathlib4-bot'] nobody
161-22673
5 months ago
206-38301
6 months ago
0-0
0 seconds
17739 Aaron1011
author:Aaron1011
feat(Topology/Order/DenselyOrdered): prove Not (IsOpen) for intervals Prove that Iic/Ici/Ioc/Ico/Icc intervals are not open in densely ordered topologies with no min/max element --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-topology merge-conflict awaiting-author 27/0 Mathlib/Topology/Order/DenselyOrdered.lean 1 8 ['github-actions', 'vihdzp'] nobody
145-5854
4 months ago
145-5854
4 months ago
0-4704
1 hour
15720 znssong
author:znssong
feat(SimpleGraph): The Bondy-Chvátal theorem The proof of the Bondy-Chvátal theorem, with Dirac's theorem and Ore's theorem as its corollary. - [x] depends on: #15536 - [ ] depends on: #15711 - [ ] depends on: #15578 new-contributor t-combinatorics merge-conflict blocked-by-other-PR 903/3 Mathlib.lean,Mathlib/Combinatorics/SimpleGraph/BondyChvatal.lean,Mathlib/Combinatorics/SimpleGraph/Finite.lean,Mathlib/Combinatorics/SimpleGraph/Hamiltonian.lean,Mathlib/Combinatorics/SimpleGraph/Path.lean,Mathlib/Combinatorics/SimpleGraph/Walk.lean,Mathlib/Dynamics/FixedPoints/Basic.lean,Mathlib/Dynamics/FixedPoints/Increasing.lean 8 3 ['github-actions', 'grunweg', 'leanprover-community-mathlib4-bot'] YaelDillies
assignee:YaelDillies
144-24940
4 months ago
144-24940
4 months ago
0-1791
29 minutes
15711 znssong
author:znssong
feat(Combinatorics/SimpleGraph): Some lemmas about walk, cycle and Hamiltonian cycle --- These lemmas are separated from the `meow-sister/BondyChvatal` branch and will be needed for the proof of the Bondy-Chvátal theorem. - [x] depends on: #15536 - [x] depends on: #16294 new-contributor t-combinatorics merge-conflict awaiting-author 407/3 Mathlib/Combinatorics/SimpleGraph/Finite.lean,Mathlib/Combinatorics/SimpleGraph/Hamiltonian.lean,Mathlib/Combinatorics/SimpleGraph/Path.lean,Mathlib/Combinatorics/SimpleGraph/Walk.lean 4 22 ['Rida-Hamadani', 'YaelDillies', 'github-actions', 'mathlib4-dependent-issues-bot', 'znssong'] nobody
144-24940
4 months ago
144-24940
4 months ago
9-13962
9 days
18629 tomaz1502
author:tomaz1502
feat(Computability.Timed): Formalization of runtime complexity of List.merge This PR adds the formalization of the runtime complexity of the merge function, defined in `Data/List/Sort`. Requires: https://github.com/leanprover-community/mathlib4/pull/15450 References: - Previous PR on mathlib3: https://github.com/leanprover-community/mathlib3/pull/14494/ - First discussion on Zulip: https://leanprover.zulipchat.com/#narrow/stream/113488-general/topic/BSc.20Final.20Project/near/220647062 - Second disussion on Zulip: https://leanprover.zulipchat.com/#narrow/stream/113488-general/topic/Formalization.20of.20Runtime.20Complexity.20of.20Sorting.20Algorithms/near/284184450 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-computability new-contributor merge-conflict awaiting-author 186/0 Mathlib.lean,Mathlib/Computability/Timed/InsertionSort.lean,Mathlib/Computability/Timed/Merge.lean 3 2 ['github-actions', 'trivial1711'] nobody
143-77259
4 months ago
143-77259
4 months ago
33-11262
33 days
19291 PieterCuijpers
author:PieterCuijpers
feat(Algebra/Order/Hom): add quantale homomorphism Definition of quantale homomorphisms as functions that are both semigroup homomorphisms and complete lattice homomorphisms. --- - [x] depends on: #19810 - [x] depends on: #19811 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra merge-conflict awaiting-author
label:t-algebra$
209/0 Mathlib.lean,Mathlib/Algebra/Order/Hom/Quantale.lean,scripts/noshake.json 3 29 ['PieterCuijpers', 'YaelDillies', 'github-actions', 'kim-em', 'mathlib4-dependent-issues-bot'] nobody
139-12518
4 months ago
139-12519
4 months ago
36-2255
36 days
20372 jvlmdr
author:jvlmdr
feat(MeasureTheory/Function): Add ContinuousLinearMap.bilinearCompLp(L) Introduce ContinuousLinearMap.bilinearCompLp and bilinearCompLpL. Generalize eLpNorm_le_eLpNorm_mul_eLpNorm theorems to include constant C in bound condition. --- Expect this may be useful for defining tempered distributions from functions in `L^p`. The definitions more or less follow `ContinuousLinearMap.compLp...`. Names are loosely analogous to `ContinuousLinearMap.bilinearComp` and `SchwartzMap.bilinLeftCLM`. Note: I preferred the spelling `hpqr : p⁻¹ + q⁻¹ = r⁻¹` with `f` in `L^p` and `g` in `L^q` to `hpqr : 1 / p = 1 / q + 1 / r`. It's easier to obtain from `ENNReal.IsConjExponent` too. A few questions: - [ ] I defined `bilinear{Left,Right}LpL` in addition to `bilinearCompLpL` because `LinearMap.mkContinuous₂` is marked as `noncomputable` and `LinearMap.mkContinuous` is not. Is this worth the extra definitions? (Note: This is not visible in the source due to `noncomputable section`.) - [ ] Should I use `C : ℝ` instead of `C : NNReal` for `eLpNorm_le_eLpNorm_mul_eLpNorm'_of_norm'`? - [ ] Is it going to be painful to have `[Fact (1 ≤ p)] [Fact (1 ≤ q)] [Fact (1 ≤ r)]`? I don't think there's a way to avoid it though. Maybe providing specialized versions for `p.IsConjExponent q` with `L^1`? Naming: - [ ] Is it satisfactory to add a `'` to the `eLpNorm_le_eLpNorm_mul_eLpNorm ` definitions in `CompareExp.lean` where `≤ ‖f x‖ * ‖g x‖` has been replaced with `≤ C * ‖f x‖ * ‖g x‖`? These could replace the existing theorems, although I don't want to break backwards compatibility. There are 5 instances: `eLpNorm_le_eLpNorm_top_mul_eLpNorm'`, `eLpNorm_le_eLpNorm_mul_eLpNorm_top'`, `eLpNorm'_le_eLpNorm'_mul_eLpNorm''`, `eLpNorm_le_eLpNorm_mul_eLpNorm_of_nnnorm'`, `eLpNorm_le_eLpNorm_mul_eLpNorm'_of_norm'` (I'm not sure why the existing theorem `eLpNorm_le_eLpNorm_mul_eLpNorm'_of_norm` has an internal `'`) - [ ] Is `bilinearLeftLpL` a suitable name? Other options: `bilinearCompLpLeftL`, `bilinearCompLeftLpL`, `bilinLeftLpL` (analogous to `SchwartzMap.bilinLeftCLM`) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-measure-probability merge-conflict 203/40 Mathlib/MeasureTheory/Function/LpSeminorm/CompareExp.lean,Mathlib/MeasureTheory/Function/LpSpace.lean 2 1 ['github-actions'] nobody
132-29866
4 months ago
132-29866
4 months ago
27-43617
27 days
17176 arulandu
author:arulandu
feat: integrals and integrability with .re Lemmas for swapping order of .re and integration/integrability. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-measure-probability merge-conflict awaiting-author 49/0 Mathlib/MeasureTheory/Function/L1Space.lean,Mathlib/MeasureTheory/Integral/IntegrableOn.lean,Mathlib/MeasureTheory/Integral/IntervalIntegral.lean,Mathlib/MeasureTheory/Integral/SetIntegral.lean 4 30 ['EtienneC30', 'arulandu', 'github-actions', 'loefflerd'] nobody
131-4299
4 months ago
131-4299
4 months ago
9-73631
9 days
14799 luigi-massacci
author:luigi-massacci
feat(Analysis/MeanInequalities): Weighted QM-AM inequality The inequality between the quadratic and arithmetic mean as a consequence of Jensen's inequality. Weighted version for positive real valued functions from a `Finset`. Fix notation for sums, switching to `∈` in place of `in`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-analysis easy merge-conflict awaiting-author 26/3 Mathlib/Analysis/MeanInequalities.lean 1 8 ['YaelDillies', 'acmepjz', 'github-actions', 'luigi-massacci', 'vihdzp'] nobody
129-83870
4 months ago
129-83870
4 months ago
0-38862
10 hours
20248 peabrainiac
author:peabrainiac
feat(Topology/Compactness): first-countable locally path-connected spaces are delta-generated Shows that all first-countable locally path-connected spaces are delta-generated (so in particular all normed spaces and convex subsets thereof are), and that delta-generated spaces are equivalently generated by the unit interval or standard simplices. --- - [ ] depends on: #21616 In principle, this should be close to all that's required to show that all simplicial complexes and CW-complexes are delta-generated; I just haven't done it yet because I'm not sure which file to best do it in. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import new-contributor t-topology merge-conflict awaiting-author blocked-by-other-PR 1189/813 Mathlib.lean,Mathlib/Geometry/Manifold/ChartedSpace.lean,Mathlib/Topology/Algebra/Module/LocallyConvex.lean,Mathlib/Topology/Compactness/DeltaGeneratedSpace.lean,Mathlib/Topology/Connected/LocPathConnected.lean,Mathlib/Topology/Connected/PathConnected.lean,Mathlib/Topology/ContinuousOn.lean,Mathlib/Topology/Homotopy/HSpaces.lean,Mathlib/Topology/Path.lean 9 22 ['YaelDillies', 'github-actions', 'kbuzzard', 'mathlib4-dependent-issues-bot', 'peabrainiac'] nobody
119-73576
3 months ago
119-73576
3 months ago
39-21495
39 days
20334 miguelmarco
author:miguelmarco
feat: allow polyrith to use a local Singular/Sage install Try to call a local install of Singular (either standalone or inside Sage) to find the witness for polyrith before trying to call the online sage cell server. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-meta merge-conflict awaiting-author 171/48 Mathlib/Tactic/Polyrith.lean,scripts/polyrith_sage.py 2 13 ['eric-wieser', 'github-actions', 'hanwenzhu', 'kim-em', 'miguelmarco'] nobody
115-38253
3 months ago
115-38253
3 months ago
27-65384
27 days
19943 AlexLoitzl
author:AlexLoitzl
feat(Computability): Add Chomsky Normal Form Grammar and translation - Define Chomsky normal form grammars - Add language-preserving translation between context-free grammars and Chomsky normal form grammars Co-authored-by: Martin Dvorak martin.dvorak@matfyz.cz --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-computability new-contributor merge-conflict awaiting-author 3151/0 Mathlib.lean,Mathlib/Computability/ChomskyNormalForm/Basic.lean,Mathlib/Computability/ChomskyNormalForm/EmptyElimination.lean,Mathlib/Computability/ChomskyNormalForm/LengthRestriction.lean,Mathlib/Computability/ChomskyNormalForm/TerminalRestriction.lean,Mathlib/Computability/ChomskyNormalForm/Translation.lean,Mathlib/Computability/ChomskyNormalForm/UnitElimination.lean,Mathlib/Computability/ContextFreeGrammar.lean 8 59 ['AlexLoitzl', 'YaelDillies', 'github-actions', 'kim-em', 'madvorak'] nobody
115-21275
3 months ago
115-21275
3 months ago
37-29014
37 days
10541 Louddy
author:Louddy
feat(Algebra/SkewMonoidAlgebra/Basic): add SkewMonoidAlgebra # Skew Monoid algebras This file presents a skewed version of `Mathlib.Algebra.MonoidAlgebra.Basic`. ## Definition We define `SkewMonoidAlgebra k G := G →₀ k` attached with a skewed convolution product. Here, the product of two elements `f g : SkewMonoidAlgebra k G` is the finitely supported function whose value at `a` is the sum of `f x * (x • g y)` over all pairs `x, y` such that `x * y = a`. This will be used in a later PR to define skew polynomial rings. Co-authored-by: María Inés de Frutos Fernández <[mariaines.dff@gmail.com](mailto:mariaines.dff@gmail.com)> --- - [x] depends on: #15878 - [x] depends on: #19084 - [ ] depends on: #22078 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra merge-conflict blocked-by-other-PR WIP
label:t-algebra$
1624/0 Mathlib.lean,Mathlib/Algebra/Group/InjSurj.lean,Mathlib/Algebra/SkewMonoidAlgebra/Basic.lean,Mathlib/Algebra/SkewMonoidAlgebra/Lift.lean 4 105 ['AntoineChambert-Loir', 'Louddy', 'YaelDillies', 'eric-wieser', 'fpvandoorn', 'github-actions', 'mariainesdff', 'mathlib4-dependent-issues-bot', 'mattrobball'] AntoineChambert-Loir
assignee:AntoineChambert-Loir
110-24901
3 months ago
110-24902
3 months ago
179-12934
179 days
21269 CharredLee
author:CharredLee
(WIP) feat (CategoryTheory/Topos): Add topos theory content This code contains basic definitions and results in topos theory, including the definition of a subobject classifier, power objects, and topoi. It is proved that every topos has exponential objects, i.e. "internal homs". The mathematical content follows chapter IV sections 1-2 of Mac Lane and Moerdijk's text "Sheaves in Geometry and Logic". --- - [x] depends on: #21281 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-category-theory merge-conflict awaiting-author WIP 1269/0 Mathlib.lean,Mathlib/CategoryTheory/Topos/Basic.lean,Mathlib/CategoryTheory/Topos/Classifier.lean,Mathlib/CategoryTheory/Topos/Exponentials.lean,Mathlib/CategoryTheory/Topos/Power.lean 5 10 ['CharredLee', 'gio256', 'github-actions', 'joelriou', 'mathlib4-dependent-issues-bot'] nobody
104-73947
3 months ago
104-73947
3 months ago
0-13879
3 hours
22245 Champitoad
author:Champitoad
feat(CategoryTheory/Subobject): add formalization of subobject classifier This introduces a file `Classifier.lean` defining the notion `Classifier C` of subobject classifier in any category `C` with a terminal object, following Section I.3 of "Sheaves in Geometry and Logic" [MM92]. This is related to but independent from #21281, because our definition associates a characteristic map to every _subobject_ rather than every _monomorphism_. Adopting this "extensional" rather than "intensional" definition allows us to formalize the proof of Proposition 1 in [MM92, Section I.3] (`hasClassifier_isRepresentable_iff`), that `C` has a subobject classifier if and only if the subobjects presheaf `sub C` is representable. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-category-theory merge-conflict awaiting-author 5219/2536 Cache/Hashing.lean,Cache/IO.lean,Cache/Lean.lean,Mathlib.lean,Mathlib/Algebra/Algebra/Defs.lean,Mathlib/Algebra/Category/AlgebraCat/Limits.lean,Mathlib/Algebra/Category/BoolRing.lean,Mathlib/Algebra/Category/FGModuleCat/Basic.lean,Mathlib/Algebra/Category/Grp/AB.lean,Mathlib/Algebra/Category/Grp/EpiMono.lean,Mathlib/Algebra/Category/HopfAlgebraCat/Monoidal.lean,Mathlib/Algebra/Category/ModuleCat/Abelian.lean,Mathlib/Algebra/Category/ModuleCat/Adjunctions.lean,Mathlib/Algebra/Category/ModuleCat/Basic.lean,Mathlib/Algebra/Category/ModuleCat/Biproducts.lean,Mathlib/Algebra/Category/ModuleCat/ChangeOfRings.lean,Mathlib/Algebra/Category/ModuleCat/Differentials/Basic.lean,Mathlib/Algebra/Category/ModuleCat/EpiMono.lean,Mathlib/Algebra/Category/ModuleCat/FilteredColimits.lean,Mathlib/Algebra/Category/ModuleCat/Kernels.lean,Mathlib/Algebra/Category/ModuleCat/Monoidal/Basic.lean,Mathlib/Algebra/Category/ModuleCat/Presheaf/Colimits.lean,Mathlib/Algebra/Category/ModuleCat/Presheaf/Limits.lean,Mathlib/Algebra/Category/ModuleCat/Subobject.lean,Mathlib/Algebra/Category/MonCat/FilteredColimits.lean,Mathlib/Algebra/Category/Ring/Colimits.lean,Mathlib/Algebra/Category/Ring/Limits.lean,Mathlib/Algebra/Group/Commute/Units.lean,Mathlib/Algebra/Group/Pointwise/Set/Card.lean,Mathlib/Algebra/Homology/ComplexShape.lean,Mathlib/Algebra/Homology/Double.lean,Mathlib/Algebra/Homology/HasNoLoop.lean,Mathlib/Algebra/Homology/Homotopy.lean,Mathlib/Algebra/Polynomial/Basic.lean,Mathlib/Algebra/Polynomial/Degree/Operations.lean,Mathlib/Algebra/Polynomial/Lifts.lean,Mathlib/Algebra/Polynomial/Sequence.lean,Mathlib/AlgebraicTopology/SimplexCategory/GeneratorsRelations/EpiMono.lean,Mathlib/Analysis/CStarAlgebra/Spectrum.lean,Mathlib/Analysis/Complex/AbelLimit.lean,Mathlib/Analysis/Complex/AbsMax.lean,Mathlib/Analysis/Complex/Angle.lean,Mathlib/Analysis/Complex/Arg.lean,Mathlib/Analysis/Complex/Basic.lean,Mathlib/Analysis/Complex/CauchyIntegral.lean,Mathlib/Analysis/Complex/Circle.lean,Mathlib/Analysis/Complex/Hadamard.lean,Mathlib/Analysis/Complex/Isometry.lean,Mathlib/Analysis/Complex/Liouville.lean,Mathlib/Analysis/Complex/LocallyUniformLimit.lean,Mathlib/Analysis/Complex/OpenMapping.lean,Mathlib/Analysis/Complex/Periodic.lean,Mathlib/Analysis/Complex/PhragmenLindelof.lean,Mathlib/Analysis/Complex/Positivity.lean,Mathlib/Analysis/Complex/Schwarz.lean,Mathlib/Analysis/Complex/UnitDisc/Basic.lean,Mathlib/Analysis/Complex/UpperHalfPlane/Exp.lean,Mathlib/Analysis/Complex/UpperHalfPlane/Metric.lean,Mathlib/Analysis/Fourier/AddCircle.lean,Mathlib/Analysis/Fourier/AddCircleMulti.lean,Mathlib/Analysis/Fourier/FourierTransformDeriv.lean,Mathlib/Analysis/Fourier/Inversion.lean,Mathlib/Analysis/Fourier/PoissonSummation.lean,Mathlib/Analysis/InnerProductSpace/TwoDim.lean,Mathlib/Analysis/MellinTransform.lean,Mathlib/Analysis/Normed/Group/Continuity.lean,Mathlib/Analysis/Normed/Lp/WithLp.lean,Mathlib/Analysis/PSeries.lean,Mathlib/Analysis/PSeriesComplex.lean,Mathlib/Analysis/SpecialFunctions/CompareExp.lean,Mathlib/Analysis/SpecialFunctions/Complex/Arctan.lean,Mathlib/Analysis/SpecialFunctions/Complex/Arg.lean,Mathlib/Analysis/SpecialFunctions/Complex/Circle.lean,Mathlib/Analysis/SpecialFunctions/Complex/Log.lean,Mathlib/Analysis/SpecialFunctions/Complex/LogBounds.lean,Mathlib/Analysis/SpecialFunctions/Exp.lean,Mathlib/Analysis/SpecialFunctions/Exponential.lean,Mathlib/Analysis/SpecialFunctions/Gamma/Basic.lean,Mathlib/Analysis/SpecialFunctions/Gamma/Beta.lean,Mathlib/Analysis/SpecialFunctions/Gamma/Deriv.lean,Mathlib/Analysis/SpecialFunctions/Gaussian/FourierTransform.lean,Mathlib/Analysis/SpecialFunctions/Gaussian/GaussianIntegral.lean,Mathlib/Analysis/SpecialFunctions/Gaussian/PoissonSummation.lean,Mathlib/Analysis/SpecialFunctions/ImproperIntegrals.lean,Mathlib/Analysis/SpecialFunctions/Integrals.lean,Mathlib/Analysis/SpecialFunctions/Log/Summable.lean,Mathlib/Analysis/SpecialFunctions/PolarCoord.lean,Mathlib/Analysis/SpecialFunctions/Pow/Asymptotics.lean,Mathlib/Analysis/SpecialFunctions/Pow/Continuity.lean,Mathlib/Analysis/SpecialFunctions/Pow/Deriv.lean,Mathlib/Analysis/SpecialFunctions/Pow/Real.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/ArctanDeriv.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Basic.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/ComplexDeriv.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Cotangent.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Series.lean,Mathlib/CategoryTheory/Abelian/FreydMitchell.lean,Mathlib/CategoryTheory/Abelian/GrothendieckAxioms/Connected.lean,Mathlib/CategoryTheory/Abelian/GrothendieckAxioms/Indization.lean,Mathlib/CategoryTheory/Abelian/GrothendieckCategory/Coseparator.lean 205 10 ['Champitoad', 'github-actions', 'joelriou'] nobody
103-83762
3 months ago
103-85035
3 months ago
0-38059
10 hours
14313 grhkm21
author:grhkm21
feat(RepresentationTheory/FdRep): FdRep is a full subcategory of Rep ``` /-- Equivalence between `FDRep` and the full subcategory of finite dimensional `Rep`. -/ def equivFiniteDimensional : FDRep k G ≌ FullSubcategory (fun V : Rep k G ↦ FiniteDimensional k V) ``` new-contributor t-algebra t-category-theory merge-conflict
label:t-algebra$
47/8 Mathlib/RepresentationTheory/FDRep.lean 1 19 ['github-actions', 'grhkm21', 'joelriou', 'kim-em', 'mathlib-bors'] nobody
101-29873
3 months ago
101-29873
3 months ago
125-12755
125 days
18626 hannahfechtner
author:hannahfechtner
feat : define Artin braid groups Define the Artin braid group on infinitely many strands. Includes a toGroup function which defines a function out of the braid group to any other group (given a function which satisfies the braid relations) (more to come in this file; next up: Artin braid groups on finitely many strands) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra merge-conflict awaiting-author
label:t-algebra$
91/0 Mathlib.lean,Mathlib/GroupTheory/SpecificGroups/BraidGroup/Basic.lean 2 22 ['github-actions', 'hannahfechtner', 'jcommelin', 'joelriou'] nobody
100-14184
3 months ago
100-14184
3 months ago
15-40648
15 days
14060 YnirPaz
author:YnirPaz
feat(SetTheory/Ordinal/Clubs): define club sets and prove basic properties Create a file where club sets are defined and their basic properties are proven. I also created a new recursion principle for ordinals, bounded recursion. --- - [ ] depends on: #19189 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-logic merge-conflict blocked-by-other-PR 315/3 Mathlib.lean,Mathlib/Order/SuccPred/Limit.lean,Mathlib/SetTheory/Cardinal/Cofinality.lean,Mathlib/SetTheory/Ordinal/Arithmetic.lean,Mathlib/SetTheory/Ordinal/Club.lean,Mathlib/SetTheory/Ordinal/Topology.lean 6 93 ['YaelDillies', 'YnirPaz', 'alreadydone', 'dupuisf', 'github-actions', 'mathlib4-dependent-issues-bot', 'vihdzp', 'zeramorphic'] nobody
97-58697
3 months ago
97-58697
3 months ago
92-44198
92 days
21959 BGuillemet
author:BGuillemet
feat(Topology/ContinuousMap): Stone-Weierstrass theorem for MvPolynomial Add the subalgebra of multivariate polynomials and prove it separates points, on the same model as `ContinuousMap/Polynomial.lean`. Prove the Stone-Weierstrass theorem and some variations for multivariate polynomials. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-topology merge-conflict 285/1 Mathlib.lean,Mathlib/Topology/ContinuousMap/MvPolynomial.lean,Mathlib/Topology/ContinuousMap/StoneWeierstrass.lean 3 1 ['github-actions'] nobody
96-15887
3 months ago
96-15887
3 months ago
16-76141
16 days
15578 znssong
author:znssong
feat(Function): Fixed points of function `f` with `f(x) >= x` We added some lemmas of fixed points of function `f` with `f(x) >= x`, where `f : α → α` is a function on a finite type `α`. This will be needed in proof of Bondy-Chvátal theorem. --- See also branch `meow-sister/BondyChvatal`. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-analysis merge-conflict awaiting-author 82/0 Mathlib.lean,Mathlib/Dynamics/FixedPoints/Basic.lean,Mathlib/Dynamics/FixedPoints/Increasing.lean 3 32 ['Ruben-VandeVelde', 'YaelDillies', 'github-actions', 'urkud', 'vihdzp', 'znssong'] nobody
88-11713
2 months ago
88-11713
2 months ago
29-48368
29 days
21018 markimunro
author:markimunro
feat(Data/Matrix): add file with key definitions and theorems about elementary row operations Prove that each elementary row operation is equivalent to a multiplication by an elementary matrix, has another row operation which inverts it, and that each elementary matrix has a left inverse. This is a very large PR and I understand it will take time. This is my first one and will likely have issues but I will be ready to answer questions/fix them as soon as possible. Co-authored-by: Christopher Lynch --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data new-contributor merge-conflict awaiting-author enhancement 1230/0 Mathlib.lean,Mathlib/Data/Matrix/ElementaryRowOperations.lean,Mathlib/Data/Matrix/GaussianElimination.lean,Mathlib/Data/Matrix/GaussianEliminationOld,Mathlib/Data/Matrix/oldnames,et --hard 18533caba32,lean-toolchain 7 n/a ['chrisflav', 'eric-wieser', 'github-actions', 'j-loreaux', 'markimunro'] nobody
69-47112
2 months ago
unknown
unknown
11768 JovanGerb
author:JovanGerb
feat: Interactive Library Rewrite This PR defines the `rw??` library rewrite tactic that uses my `RefinedDiscrTree`. This is a point&click tactic, letting the user click on subexpressions in the main goal. The results are sorted by relevance, and are separated into sections based on the matched pattern. It comes with a filter button that allows you to switch between the (default) filtered view, with removed duplicate lemmas and not showing lemma names, and the complete view. There is also a section for definitionally unfolding the selected expression - these rewrites do not correspond to a library lemma. --- - [ ] depends on: #11968 - [x] depends on: #12016 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-meta merge-conflict blocked-by-other-PR 2788/1253 Mathlib.lean,Mathlib/Lean/GoalsLocation.lean,Mathlib/Lean/Meta/RefinedDiscrTree.lean,Mathlib/Lean/Meta/RefinedDiscrTree/Basic.lean,Mathlib/Lean/Meta/RefinedDiscrTree/Encode.lean,Mathlib/Lean/Meta/RefinedDiscrTree/Initialize.lean,Mathlib/Lean/Meta/RefinedDiscrTree/Lookup.lean,Mathlib/Lean/Meta/RefinedDiscrTree/Pi.lean,Mathlib/Tactic.lean,Mathlib/Tactic/FunProp.lean,Mathlib/Tactic/FunProp/Elab.lean,Mathlib/Tactic/FunProp/StateList.lean,Mathlib/Tactic/FunProp/Theorems.lean,Mathlib/Tactic/FunProp/Types.lean,Mathlib/Tactic/Widget/InteractiveUnfold.lean,Mathlib/Tactic/Widget/LibraryRewrite.lean,Mathlib/Topology/Defs/Basic.lean,MathlibTest/LibraryRewrite.lean,MathlibTest/RefinedDiscrTree.lean,scripts/noshake.json 20 n/a ['JovanGerb', 'eric-wieser', 'fpvandoorn', 'github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot'] nobody
68-28146
2 months ago
unknown
unknown
15212 victorliu5296
author:victorliu5296
feat: Add fundamental theorem of calculus-2 for Banach spaces add the Mean Value Theorem for Banach spaces to the library and include reference for the theorem statement This theorem states that if `f : X → Y` is differentiable along the line segment from `a` to `b`, then the change in `f` equals the integral of its derivative along this path. This extends the mean value theorem to Banach spaces. This can be used for the eventual proof of the Newton-Kantorovich theorem with 1 constant contained inside the added reference. Here is the discussion on Zulipchat: https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/Contributing.20FTC-2.20for.20Banach.20spaces new-contributor t-measure-probability t-analysis merge-conflict awaiting-author 60/1 Mathlib/MeasureTheory/Integral/FundThmCalculus.lean 1 3 ['github-actions', 'hrmacbeth', 'victorliu5296'] nobody
64-42101
2 months ago
64-42101
2 months ago
51-85104
51 days
22701 ctchou
author:ctchou
feat(Combinatorics): the Katona circle method This file formalizes the Katona circle method. From PlainCombi (LeanCamCombi): https://github.com/YaelDillies/LeanCamCombi/blob/master/LeanCamCombi/PlainCombi/KatonaCircle.lean Co-authored-by: Yaël Dillies new-contributor t-combinatorics merge-conflict 121/0 Mathlib.lean,Mathlib/Combinatorics/KatonaCircle.lean 2 1 ['github-actions'] nobody
63-78056
2 months ago
63-78056
2 months ago
30-8337
30 days
21488 imbrem
author:imbrem
feat(CategoryTheory/Monoidal): premonoidal categories Add support for premonoidal categories --- Still want to add support for: - Premonoidal braided/symmetric categories - The monoidal coherence theorem, which I've already ported in my `discretion` library - The `coherence` tactic, which should work fine for premonoidal categories too but wanted to get this in front of reviewers ASAP to make sure my general approach was alright [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-category-theory merge-conflict 900/361 Mathlib/Algebra/Category/ModuleCat/Presheaf/Monoidal.lean,Mathlib/CategoryTheory/Bicategory/End.lean,Mathlib/CategoryTheory/GradedObject/Monoidal.lean,Mathlib/CategoryTheory/Localization/Monoidal.lean,Mathlib/CategoryTheory/Monoidal/Braided/Basic.lean,Mathlib/CategoryTheory/Monoidal/Category.lean,Mathlib/CategoryTheory/Monoidal/Center.lean,Mathlib/CategoryTheory/Monoidal/CoherenceLemmas.lean,Mathlib/CategoryTheory/Monoidal/Discrete.lean,Mathlib/CategoryTheory/Monoidal/End.lean,Mathlib/CategoryTheory/Monoidal/Free/Basic.lean,Mathlib/CategoryTheory/Monoidal/Functor.lean,Mathlib/CategoryTheory/Monoidal/FunctorCategory.lean,Mathlib/CategoryTheory/Monoidal/Mon_.lean,Mathlib/CategoryTheory/Monoidal/Opposite.lean,Mathlib/CategoryTheory/Monoidal/Transport.lean,Mathlib/Tactic/CategoryTheory/Monoidal/Datatypes.lean,Mathlib/Tactic/CategoryTheory/Monoidal/Normalize.lean,Mathlib/Tactic/CategoryTheory/Monoidal/PureCoherence.lean,Mathlib/Tactic/CategoryTheory/MonoidalComp.lean,MathlibTest/StringDiagram.lean 21 9 ['YaelDillies', 'github-actions', 'grunweg', 'imbrem', 'kim-em', 'leanprover-community-bot-assistant'] nobody
61-24289
2 months ago
61-24290
2 months ago
58-20339
58 days
20873 vbeffara
author:vbeffara
feat(Topology/Covering): path lifting and homotopy lifting This proves the existence and uniqueness of path and homotopy lifts through covering maps. --- I tried to separate as much of the proof as possible into separate PRs (which are already in Mathlib now), but the proof here relies on a monolithic construction of an explicit lift along a well-chosen subdivision, in `partial_lift`, with associated definitions. Only one standalone lean file added. An older WIP PR #10084 by Junyan Xu @alreadydone proves similar results using a very similar construction for path lifting, with a different argument to obtain continuity for homotopy lifting. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-topology merge-conflict awaiting-author 281/1 Mathlib.lean,Mathlib/Topology/Covering/Basic.lean,Mathlib/Topology/Covering/Lift.lean 3 9 ['alreadydone', 'github-actions', 'grunweg', 'vbeffara'] nobody
60-27017
1 month ago
60-27017
1 month ago
55-53553
55 days
20313 thefundamentaltheor3m
author:thefundamentaltheor3m
feat(Data/Complex/Exponential): prove some useful results about the complex exponential. This PR proves two basic results about the complex exponential: * `abs_exp_mul_I (x : ℂ) : abs (Complex.exp (I * x)) = Real.exp (-x.im)` * `one_sub_rexp_re_le_abs_one_sub_cexp (x : ℂ) : 1 - Real.exp x.re ≤ Complex.abs (1 - Complex.exp x)` Both results were proved as part of the sphere packing project. There's a chance they're too specific for mathlib, but I thought they were worth PRing anyway. Would it also be a good idea to tag `abs_exp_mul_I` with `simp`? Feedback/suggestions welcome. Note: `one_sub_rexp_re_le_abs_one_sub_cexp` was proved by Bhavik Mehta @b-mehta --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-analysis merge-conflict 167/141 Mathlib.lean,Mathlib/Analysis/Complex/Basic.lean,Mathlib/Analysis/SpecialFunctions/Log/ERealExp.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Chebyshev.lean,Mathlib/Data/Complex/Exponential/Defs.lean,Mathlib/Data/Complex/Exponential/Lemmas.lean,Mathlib/Data/Complex/ExponentialBounds.lean,Mathlib/Tactic/FunProp.lean,MathlibTest/Recall.lean,MathlibTest/positivity.lean 10 12 ['b-mehta', 'github-actions', 'kim-em', 'thefundamentaltheor3m', 'trivial1711'] nobody
52-84615
1 month ago
52-84615
1 month ago
25-60481
25 days
20730 kuotsanhsu
author:kuotsanhsu
feat(LinearAlgebra/Matrix/SchurTriangulation): prove Schur decomposition/triangulation `Matrix.schur_triangulation` shows that a matrix over an algebraically closed field is unitarily similar to an upper triangular matrix --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra merge-conflict awaiting-author
label:t-algebra$
317/2 Mathlib.lean,Mathlib/LinearAlgebra/Matrix/Block.lean,Mathlib/LinearAlgebra/Matrix/SchurTriangulation.lean,Mathlib/Logic/Equiv/Basic.lean 4 14 ['eric-wieser', 'github-actions', 'kim-em', 'kuotsanhsu'] nobody
52-80747
1 month ago
52-80747
1 month ago
13-60072
13 days
15654 TpmKranz
author:TpmKranz
feat(Computability): language-preserving maps between NFA and RE Map REs to NFAs via Thompson's construction and NFAs to REs using GNFAs Last chunk of #12648 --- - [ ] depends on: #15651 - [ ] depends on: #15649 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-zulip t-computability new-contributor merge-conflict blocked-by-other-PR 985/2 Mathlib.lean,Mathlib/Computability/GNFA.lean,Mathlib/Computability/Language.lean,Mathlib/Computability/NFA.lean,Mathlib/Computability/RegularExpressions.lean,Mathlib/Data/FinEnum/Option.lean,docs/references.bib 7 3 ['github-actions', 'leanprover-community-mathlib4-bot', 'meithecatte'] nobody
34-77865
1 month ago
34-77870
1 month ago
0-179
2 minutes
23338 WilliamCoram
author:WilliamCoram
feat: restricted power series form a ring We define restricted powerseries over a normed ring R, and show they form a ring when R has the ultrametric property. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-number-theory merge-conflict 186/0 Mathlib.lean,Mathlib/RingTheory/PowerSeries/Restricted.lean 2 18 ['Paul-Lez', 'WilliamCoram', 'github-actions', 'grunweg', 'leanprover-community-bot-assistant'] nobody
26-33783
26 days ago
26-33785
26 days ago
48-76736
48 days
13685 niklasmohrin
author:niklasmohrin
feat(Combinatorics): add definitions for network flows Although we might not have any super-interesting results ready for mathlib yet, I feel that the definitions from this commit are already mature enough to include. These definitions are ported from last semester's work we did at https://github.com/niklasmohrin/lean-seminar-2023 and I have put some time in to refactor our code to `Int` and now to any parameter `R`. In the linked repository, there is some more stuff that I can send in. One obstacle without integer values is that it is not clear why a maximum flow would exist. I think the best way to tackle this would be to prove max-flow-min-cut theorem and implement the Ford-Fulkerson algorithm. It has been pointed out on Zulip that there is an [Isabelle formalization of the Edmonds Karp Algorithm](https://www.isa-afp.org/entries/EdmondsKarp_Maxflow.html). I feel that the definitions are pretty solid and it makes sense to include them, even if just for unifying definitions across downstream projects. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-combinatorics merge-conflict awaiting-author 244/0 Mathlib.lean,Mathlib/Combinatorics/Flow/Basic.lean,docs/references.bib 3 57 ['Shreyas4991', 'YaelDillies', 'b-mehta', 'github-actions', 'leanprover-community-bot-assistant', 'madvorak', 'niklasmohrin'] nobody
25-70063
25 days ago
25-70065
25 days ago
86-21072
86 days
21603 imbrem
author:imbrem
feat(CategoryTheory/ChosenFiniteProducts): add basic ChosenFiniteCoproducts class Added basic `ChosenFiniteCoproducts` class, and started porting some of the lemmas about `ChosenFiniteProducts` suitably translated --- This, combined with #20182 modified to use chosen finite coproducts and premonoidal categories (#21488), should be enough for me to formalize strong Elgot categories, and hence a lot of categorical iteration theory for my PhD thesis. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-category-theory merge-conflict awaiting-author 261/2 Mathlib/CategoryTheory/ChosenFiniteProducts.lean 1 17 ['TwoFX', 'YaelDillies', 'github-actions', 'grunweg', 'imbrem', 'joelriou', 'leanprover-community-bot-assistant'] TwoFX and joelriou
assignee:TwoFX assignee:joelriou
25-2480
25 days ago
25-2662
25 days ago
89-21170
89 days
22639 b-reinke
author:b-reinke
feat(Mathlib/GroupTheory/FreeGroup): theory of (cyclically) reduced words Upstreamed from the [EquationalTheories](https://github.com/teorth/equational_theories) project. This PR defines in the new file `Mathlib/GroupTheory/FreeGroup/ReducedWords.lean` some extra lemmas for free groups, in particular about (cyclically) reduced words. ## Main declarations * `FreeGroup.Red.reduced`: the predicate for reduced words * `FreeGroup.Red.cyclicallyReduced`: the predicate for cyclically reduced words ## Main statements * `FreeGroup.infinite_order`: nontrivial elements of a free group have infinite order * `FreeGroup.zpow_left_injective`: taking n-th powers is an injective function on the free group Co-authored-by: Amir Livne Bar-on - [ ] depends on: #23366 - [ ] depends on: #23367 - [ ] depends on: #23368 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra merge-conflict blocked-by-other-PR
label:t-algebra$
429/0 Mathlib.lean,Mathlib/GroupTheory/FreeGroup/Basic.lean,Mathlib/GroupTheory/FreeGroup/Reduce.lean,Mathlib/GroupTheory/FreeGroup/ReducedWords.lean 4 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
24-45371
24 days ago
24-45374
24 days ago
20-75471
20 days
15651 TpmKranz
author:TpmKranz
feat(Computability/NFA): operations for Thompson's construction Lays the groundwork for a proof of equivalence of RE and NFA, w.r.t. described language. Actual connection to REs comes later, after the groundwork for the opposite direction has been laid. Third chunk of #12648 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-zulip t-computability new-contributor merge-conflict awaiting-author 307/5 Mathlib/Computability/NFA.lean 1 15 ['TpmKranz', 'YaelDillies', 'dupuisf', 'github-actions', 'leanprover-community-bot-assistant', 'meithecatte'] nobody
21-14071
21 days ago
21-14072
21 days ago
45-84611
45 days
22361 rudynicolop
author:rudynicolop
feat(Computability/NFA): nfa closure properties Add the closure properties union, intersection and reversal for NFA. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-zulip t-computability new-contributor merge-conflict awaiting-author 218/2 Mathlib/Computability/Language.lean,Mathlib/Computability/NFA.lean 2 90 ['EtienneC30', 'b-mehta', 'github-actions', 'leanprover-community-bot-assistant', 'meithecatte', 'rudynicolop'] EtienneC30
assignee:EtienneC30
21-13145
21 days ago
21-13147
21 days ago
39-67601
39 days
23349 BGuillemet
author:BGuillemet
feat: add LocallyLipschitzOn.lipschitzOnWith_of_isCompact and two small lemmas about Lipschitz functions Main feat (in Mathlib/Topology/EMetricSpace/Basic.lean): if a function `f` from an extended pseudometric space to a pseudometric space is locally Lipschitz on a compact subset `s`, then `f` is Lipschitz on `s`. The theorem is true only when the codomain of `f` is a pseudometric space, so it needs imports from Mathlib/Topology/MetricSpace. Other small feat (in Mathlib/Analysis/Calculus/ContDiff/RCLike.lean): a function that is continuously differentiable on an open subset is locally Lipschitz on this subset. --- - [ ] depends on: #22890 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import new-contributor t-topology merge-conflict 59/4 Mathlib/Analysis/Calculus/ContDiff/RCLike.lean,Mathlib/Topology/EMetricSpace/Lipschitz.lean 2 4 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] PatrickMassot
assignee:PatrickMassot
13-9385
13 days ago
13-9387
13 days ago
35-30364
35 days

PRs not into the master branch

Number Author Title Description Labels +/- Modified files (first 100) 📝 💬 All users who commented or reviewed Assignee(s) Updated Last status change total time in review
18472 FR-vdash-bot
author:FR-vdash-bot
perf: lower the priority of `Comm*.to*` instances `CommRing.toRing` is an exception. `CommRing` is so important that it needs to be looked up early. An important goal of #7873 is also to search for `Zero/One/Add/Mul` instances first along `Zero/One/Add/Mul` -> ... -> `Ring` -> `CommRing` -> `Field`. --- - [ ] depends on: #18474 - [ ] depends on: #18641 From #7873. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-bench slow-typeclass-synthesis t-algebra blocked-by-other-PR
label:t-algebra$
33/10 Mathlib/Algebra/Group/Defs.lean,Mathlib/Algebra/GroupWithZero/Defs.lean,Mathlib/Algebra/Ring/Defs.lean,Mathlib/AlgebraicGeometry/Cover/Open.lean,Mathlib/Data/Int/Cast/Defs.lean,Mathlib/Data/Nat/Cast/Defs.lean,Mathlib/LinearAlgebra/Matrix/Charpoly/Coeff.lean,Mathlib/NumberTheory/LegendreSymbol/GaussEisensteinLemmas.lean,Mathlib/NumberTheory/NumberField/Discriminant/Defs.lean,Mathlib/NumberTheory/Padics/PadicNumbers.lean,Mathlib/NumberTheory/Zsqrtd/QuadraticReciprocity.lean,Mathlib/RingTheory/Filtration.lean,Mathlib/RingTheory/Localization/Integral.lean,Mathlib/Topology/MetricSpace/Polish.lean 14 5 ['FR-vdash-bot', 'github-actions', 'leanprover-bot', 'mathlib4-dependent-issues-bot'] nobody
214-78489
7 months ago
215-3668
7 months ago
0-258
4 minutes
18464 FR-vdash-bot
author:FR-vdash-bot
perf: lower the priority of `toMul` and `toAdd` instances A subsequent PR will try to swap the priorities of `Semigroup.toMul` and `MulOneClass.toMul` to see if it gets better. --- - [ ] depends on: #18472 From #7873. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-bench slow-typeclass-synthesis t-algebra blocked-by-other-PR
label:t-algebra$
38/12 Mathlib/Algebra/BigOperators/Ring/List.lean,Mathlib/Algebra/Group/Defs.lean,Mathlib/Algebra/GroupWithZero/Defs.lean,Mathlib/Algebra/Ring/Defs.lean,Mathlib/Algebra/Ring/Ext.lean 5 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
214-62502
7 months ago
221-74724
7 months ago
0-8515
2 hours
18706 FR-vdash-bot
author:FR-vdash-bot
perf: change the priority of `*.toSemiring` instances Need to fix some regressions in subsequent PRs. --- - [ ] depends on: #18468 - [ ] depends on: #18470 From #7873. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-bench slow-typeclass-synthesis t-algebra blocked-by-other-PR WIP
label:t-algebra$
24/15 Mathlib/Algebra/Field/Defs.lean,Mathlib/Algebra/Order/Kleene.lean,Mathlib/Algebra/Ring/Defs.lean,Mathlib/FieldTheory/Extension.lean,Mathlib/FieldTheory/PurelyInseparable.lean,Mathlib/LinearAlgebra/Matrix/Charpoly/Coeff.lean,Mathlib/RingTheory/Etale/Field.lean,Mathlib/RingTheory/Filtration.lean,Mathlib/RingTheory/Localization/Integral.lean 9 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
59-998
1 month ago
214-63136
7 months ago
0-576
9 minutes
18641 FR-vdash-bot
author:FR-vdash-bot
perf: change the priority of `*.toRing` instances --- - [ ] depends on: #18468 - [ ] depends on: #18470 From #7873. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-bench slow-typeclass-synthesis t-algebra blocked-by-other-PR
label:t-algebra$
7/1 Mathlib/Algebra/Field/Defs.lean,Mathlib/Algebra/Ring/BooleanRing.lean,Mathlib/Algebra/Ring/Defs.lean,Mathlib/RingTheory/Valuation/ValuationSubring.lean 4 5 ['FR-vdash-bot', 'github-actions', 'leanprover-bot', 'mathlib4-dependent-issues-bot'] nobody
59-996
1 month ago
216-54247
7 months ago
0-627
10 minutes
24543 pfaffelh
author:pfaffelh
feat (Topology/Compactness/CompactSystem): Set system of finite unions of sets in a compact system is again a compact system feat (Topology/Compactness/CompactSystem): The set system of finite unions of sets in a compact system is a compact system A compact system is a set system with the following property: If all finite intersections of a sequence in the set system is non-empty, the countable intersection is not empty. Starting with a compact system, consider the finite unions of sets in the copact system. Such sets again form a compact system (`IsCompactSystem.union.isCompactSystem`). --- - [x] depends on: #24541 - [x] depends on: #24542 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-topology blocked-by-other-PR 431/2 Mathlib/Topology/Compactness/CompactSystem.lean 1 4 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
7-82487
7 days ago
7-82487
7 days ago
0-1830
30 minutes
24542 pfaffelh
author:pfaffelh
feat (Topology/Compactness/CompactSystem): Closed and compact square cylinders form a compact system. feat (Topology/Compactness/CompactSystem): Closed and compact square cylinders form a compact system. A square cylinder is a set of the form `s.pi t` in a product space. A closed compact square cylinder has `IsClosed (t i)` and `IsCompact (t i)` for all `i ∈ s`. This set system is a compact system (as introduced in PR #24541). Streamline the definition of square cylinders in MeasureTheory/Constructions/Cylinders on the way. Co-authors: Rémy Degenne remy.degenne@inria.fr --- - [x] depends on: #24541 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-topology blocked-by-other-PR 264/66 Mathlib/Data/Set/Prod.lean,Mathlib/MeasureTheory/Constructions/Cylinders.lean,Mathlib/MeasureTheory/Constructions/ProjectiveFamilyContent.lean,Mathlib/Topology/Compactness/CompactSystem.lean 4 4 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
0-80012
22 hours ago
0-84878
23 hours ago
0-192
3 minutes
13158 erdOne
author:erdOne
refactor(RingTheory/OreLocalization/Module): remove `LocalizedModule.mk`. --- - [x] depends on: #13151 - [ ] depends on: #13156 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict blocked-by-other-PR
label:t-algebra$
49/48 Mathlib/RingTheory/OreLocalization/Basic.lean,Mathlib/RingTheory/OreLocalization/Module.lean 2 1 ['leanprover-community-mathlib4-bot'] nobody
335-23447
11 months ago
335-23470
11 months ago
0-0
0 seconds
11156 smorel394
author:smorel394
feat(LinearAlgebra/{TensorProductBasis,Dual}): basis and dual of `PiTensorProduct` Construct a basis of a `PiTensorProduct` of modules given bases of the modules, and relationship between the dual of a `PiTensorProduct` and the `PiTensorProduct` of the duals. Main results: * `Basis.piTensorProduct` (in `LinearAlgebra/TensorProductBasis.lean`): Let `ι` be a `Fintype` and `M` be a family of modules indexed by `ι`. If `b i : κ i → M i` is a basis for every `i` in `ι`, then `fun (p : Π i, κ i) ↦ ⨂ₜ[R] i, b i (p i)` is a basis of `⨂[R] i, M i`. * `PiTensorProduct.dualDistrib` (in `LinearAlgebra/Dual.lean`): The canonical linear map from `⨂[R] i, Dual R (M i)` to `Dual R (⨂[R] i, M i)`, sending `⨂ₜ[R] i, f i` to the composition of `PiTensorProduct.map f` with the linear equivalence `⨂[R] i, R →ₗ R` given by multiplication. * `PiTensorProduct.dualDistribEquiv` (also in `LinearAlgebra/Dual.lean`): A linear equivalence between `⨂[R] i, Dual R (M i)` and `Dual R (⨂[R] i, M i)` when all `M i` are finite free modules. If `f : (i : ι) → Dual R (M i)`, then this equivalence sends `⨂ₜ[R] i, f i` to the composition of `PiTensorProduct.map f` with the natural isomorphism `⨂[R] i, R ≃ R` given by multiplication. - [ ] depends on: #11155 (currently used as the base branch; do not merge without switching it back to `master`!) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import new-contributor t-algebra merge-conflict please-adopt blocked-by-other-PR
label:t-algebra$
166/2 Mathlib/LinearAlgebra/DirectSum/Finsupp.lean,Mathlib/LinearAlgebra/Dual.lean,Mathlib/LinearAlgebra/TensorProduct/Basis.lean 3 4 ['eric-wieser', 'github-actions', 'leanprover-community-mathlib4-bot'] nobody
161-22673
5 months ago
206-38301
6 months ago
0-0
0 seconds
23644 JovanGerb
author:JovanGerb
Lean pr testing 7804 Testing an optimization in `simp` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict 4/4 lake-manifest.json,lakefile.lean,lean-toolchain 3 3 ['github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot'] nobody
4-29888
4 days ago
66-75572
2 months ago
0-2933
48 minutes
24808 JovanGerb
author:JovanGerb
lean pr testing 8294 Testing a cache optimization in `isDefEq`, to avoid exponential blowup during unification. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict 243/98 Mathlib.lean,Mathlib/Algebra/BigOperators/Group/Finset/Basic.lean,Mathlib/Algebra/BigOperators/Group/Finset/Preimage.lean,Mathlib/Algebra/BigOperators/Intervals.lean,Mathlib/Algebra/Group/Submonoid/Basic.lean,Mathlib/Algebra/GroupWithZero/Basic.lean,Mathlib/Algebra/GroupWithZero/Defs.lean,Mathlib/Algebra/GroupWithZero/NeZero.lean,Mathlib/Algebra/Homology/DifferentialObject.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Affine/Formula.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Affine/Point.lean,Mathlib/Analysis/Complex/ValueDistribution/CharacteristicFunction.lean,Mathlib/Analysis/InnerProductSpace/Spectrum.lean,Mathlib/Analysis/LConvolution.lean,Mathlib/Analysis/NormedSpace/Alternating/Curry.lean,Mathlib/CategoryTheory/Limits/VanKampen.lean,Mathlib/Data/Finset/Fold.lean,Mathlib/Data/Finset/Image.lean,Mathlib/Data/Int/Init.lean,Mathlib/Data/Matrix/Mul.lean,Mathlib/Data/Nat/Factorization/Basic.lean,Mathlib/Data/Set/Function.lean,Mathlib/Data/Set/Image.lean,Mathlib/Data/Vector/MapLemmas.lean,Mathlib/Data/ZMod/Basic.lean,Mathlib/MeasureTheory/Group/Convolution.lean,Mathlib/MeasureTheory/Group/IntegralConvolution.lean,Mathlib/NumberTheory/ArithmeticFunction.lean,Mathlib/NumberTheory/Divisors.lean,Mathlib/Probability/Distributions/Gaussian/Real.lean,Mathlib/Topology/Algebra/InfiniteSum/NatInt.lean,Shake/Main.lean,lake-manifest.json,lakefile.lean,lean-toolchain 35 21 ['JovanGerb', 'adomani', 'github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot'] nobody
2-686
2 days ago
2-686
2 days ago
0-11360
3 hours

PRs from a fork of mathlib

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
23772 SEU-Prime
author:SEU-Prime
Create Amice.lean i built amice equiv [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-number-theory WIP 283/0 Mathlib/NumberTheory/Padics/Amice.lean 1 2 ['grunweg'] nobody
63-21594
2 months ago
63-21594
2 months ago
0-0
0 seconds
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/) will-close-soon t-algebra
label:t-algebra$
17/0 Mathlib/FieldTheory/RatFunc/Basic.lean 1 1 ['joneugster'] nobody
52-80776
1 month ago
52-80776
1 month ago
0-0
0 seconds
25516 kim-em
author:kim-em
chore: test PR from fork This PR tests making a PR from a fork. 1/0 Mathlib/Computability/AkraBazzi/AkraBazzi.lean 1 1 ['bryangingechen'] nobody
3-22035
3 days ago
3-58538
3 days ago
0-0
0 seconds
25537 literandltx
author:literandltx
feat(number_theory/legendre_symbol): Add sqrt‐of‐residue theorems for p=4k+3 and p=8k+5 Add a new file `QuadraticResidueRoots.lean` under `Mathlib/NumberTheory/LegendreSymbol/` that proves two explicit “square-root of quadratic residue” theorems for primes of the specific form. - **`exists_sqrt_of_residue_mod4_eq3`** for primes `p = 4*k + 3` - **`exists_sqrt_of_residue_mod8_eq5`** for primes `p = 8*k + 5` It also introduces the helper lemmas `euler_criterion_traditional` and `legendreSym.at_two_mod8_eq_5`. Import lines in `Mathlib.lean` and `Mathlib/NumberTheory/LegendreSymbol/Basic.lean` have been updated accordingly. new-contributor 217/0 Mathlib.lean,Mathlib/NumberTheory/LegendreSymbol/Basic.lean,Mathlib/NumberTheory/LegendreSymbol/QuadraticReciprocity.lean,Mathlib/NumberTheory/LegendreSymbol/QuadraticResidueRoots.lean 4 0 [] nobody
3-19735
3 days ago
3-19735
3 days ago
0-0
0 seconds
25599 adomani
author:adomani
test: autolabel from forks --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) test-ci awaiting-author WIP 1/1 Mathlib/Tactic/Eval.lean,newFileOnMaster.md 2 3 ['adomani', 'bryangingechen', 'github-actions'] nobody
0-33809
9 hours ago
1-9271
1 day ago
0-0
0 seconds
25623 mattrobball
author:mattrobball
feat: decidable equality for `Quiver.Path` Given a quiver with decidable equality on its vertices and arrows, we construct an instance of decidable equality for `Quiver.Path`. We proceed through a recursion on the length of the path utilizing an intermediate subtype of uniformly bounded paths `Quiver.Path.BoundedPath`. This was motivated by doing computations on small quivers with Lean. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 69/0 Mathlib/Combinatorics/Quiver/Path.lean 1 1 ['github-actions'] nobody
0-22514
6 hours ago
0-22603
6 hours ago
0-0
0 seconds
3610 TimothyGu
author:TimothyGu
feat: derive Infinite automatically for inductive types Deals with recursive types, but not mutually recursive types or types with indices right now. See docstring for details. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta merge-conflict awaiting-author 517/0 Mathlib.lean,Mathlib/Tactic/DeriveInfinite.lean,test/DeriveInfinite.lean 3 11 ['TimothyGu', 'digama0', 'eric-wieser', 'grunweg', 'kim-em', 'kmill'] kmill
assignee:kmill
155-56406
5 months ago
155-56406
5 months ago
0-0
0 seconds

PRs with an 'approved' review

Number Author Title Description Labels +/- Modified files (first 100) 📝 💬 All users who commented or reviewed Assignee(s) Approval(s) Updated Last status change total time in review
9352 chenyili0818
author:chenyili0818
feat: arithmetic lemmas for `gradient` This file is based on Mathlib.Analysis.Calculus.Gradient.Basic, and describes the calculation properties Co-authored-by: Ziyu Wang [tropicalfish910@gmail.com](mailto:tropicalfish910@gmail.com) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis awaiting-author 404/0 Mathlib.lean,Mathlib/Analysis/Calculus/Gradient/Lemmas.lean 2 30 ['chenyili0818', 'github-actions', 'jcommelin', 'sgouezel', 'winstonyin'] nobody 1
313-42767
10 months ago
475-23932
1 year ago
51-80670
51 days
11890 adomani
author:adomani
feat: the terminal refine linter A linter that warns on usages of `refine` and `refine'` as a finishing tactic. See this [Zulip discussion](https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/Usage.20of.20refine'). ### Conclusion of the experiment Systematic replacements of terminal `refine` with `exact` leads to an overall slow-down. --- - [ ] depends on: #15616 (disable the linter in downstream projects) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-linter awaiting-author 77/0 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter/TerminalRefineLinter.lean 3 14 ['adomani', 'github-actions', 'grunweg', 'joneugster', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'urkud'] nobody 1
294-43251
9 months ago
294-43253
9 months ago
18-13508
18 days
15809 archiebrowne
author:archiebrowne
feat(RingTheory/MvPolynomial/Ideal): introduce new lemmas about MvPolynomial Ideals Four new lemmas about MvPolynomialIdeals `sub_span_span_sub`, `span_eq_iff_basis_sub`, `mem_basis_mem_span`, `mem_span_exists_dvd_mem_basis`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra awaiting-author
label:t-algebra$
38/0 Mathlib/RingTheory/MvPolynomial/Ideal.lean 1 6 ['Ruben-VandeVelde', 'github-actions', 'riccardobrasca'] riccardobrasca
assignee:riccardobrasca
1
203-16688
6 months ago
258-18608
8 months ago
41-7533
41 days
18461 hannahfechtner
author:hannahfechtner
feat: left and right common multiples mixins add mixins for left and right common multiples. These carry the data of what factors are used to create the common multiples --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra awaiting-author
label:t-algebra$
78/0 Mathlib/Algebra/Group/Defs.lean 1 13 ['github-actions', 'hannahfechtner', 'jcommelin', 'kbuzzard', 'kim-em', 'trivial1711'] nobody 1
140-38439
4 months ago
140-38439
4 months ago
69-35596
69 days
22320 jjdishere
author:jjdishere
feat(RingTheory/WittVector): the Teichmuller series In this PR, we show that every element `x` of the Witt vectors `𝕎 R` can be written as the (`p`-adic) summation of the Teichmuller series. Instead of using `tsum`, we only show that `p ^ (n + 1)` divides `x` minus the summation of the first `n + 1` terms of the Teichmuller series. We also show that if `p` divides the first (n + 1) coefficients of a Witt vector, then `p^(n+1)` divides the `n`-th ghost component. #21564 depends on this PR. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra awaiting-author
label:t-algebra$
204/2 Mathlib.lean,Mathlib/Algebra/Ring/Aut.lean,Mathlib/FieldTheory/Perfect.lean,Mathlib/RingTheory/WittVector/Basic.lean,Mathlib/RingTheory/WittVector/Complete.lean,Mathlib/RingTheory/WittVector/TeichmullerSeries.lean 6 12 ['github-actions', 'jjdishere', 'riccardobrasca'] nobody 1
97-25322
3 months ago
97-25322
3 months ago
6-3646
6 days
22159 shetzl
author:shetzl
feat: add definition of pushdown automata Add the definition of pushdown automata and their two acceptance conditions: acceptance based on empty stack and acceptance based on final state. Co-authored-by: Tobias Leichtfried --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-computability new-contributor awaiting-author 70/0 Mathlib.lean,Mathlib/Computability/PDA.lean 2 34 ['YaelDillies', 'github-actions', 'madvorak', 'shetzl'] nobody 1
84-38789
2 months ago
84-38789
2 months ago
20-81771
20 days
24218 alreadydone
author:alreadydone
chore(Algebra): remove `mid_assoc` from `IsMulCentral` as it is a consequence of left and right associativity in the presence of commutativity. Also change the commutativity condition to use `Commute`. --- Even without commutativity, left and right associativity of an element `e` in a magma is sufficient to prove that elements of the form `e * x * e` (the "corner" of `e`) form a submagma. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
31/69 Mathlib/Algebra/Algebra/NonUnitalSubalgebra.lean,Mathlib/Algebra/Group/Center.lean,Mathlib/Algebra/GroupWithZero/Center.lean,Mathlib/Algebra/Ring/Center.lean,Mathlib/Algebra/Ring/CentroidHom.lean,Mathlib/Algebra/Star/Center.lean,Mathlib/Algebra/Star/CentroidHom.lean,Mathlib/GroupTheory/Submonoid/Center.lean,Mathlib/LinearAlgebra/Basis/Submodule.lean,Mathlib/LinearAlgebra/QuadraticForm/Basic.lean,Mathlib/RingTheory/Idempotents.lean,Mathlib/RingTheory/NonUnitalSubsemiring/Basic.lean 12 8 ['alreadydone', 'github-actions', 'mans0954'] nobody 1
50-12169
1 month ago
50-27229
1 month ago
50-27219
50 days
18210 vihdzp
author:vihdzp
feat(Order/Hom/Basic): `WithBot (Fin n) ≃o Fin (n + 1)` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order awaiting-author 16/0 Mathlib/Order/Hom/Basic.lean 1 8 ['Command-Master', 'Ruben-VandeVelde', 'github-actions', 'urkud', 'vihdzp'] nobody 2
45-69064
1 month ago
216-73142
7 months ago
10-77913
10 days
24036 Louddy
author:Louddy
feat: add `HeightOneSpectrum.ofPrime` Add a definition relating elements of type `HeightOneSpectrum R` with the (nonzero) prime elements of the monoid with zero `Ideal R`. (Note the distinction between `Prime` and `Ideal.IsPrime`). The documentation string is inspired from [Ideal.prime_iff_isPrime](https://leanprover-community.github.io/mathlib4_docs/Mathlib/RingTheory/DedekindDomain/Ideal.html#Ideal.prime_iff_isPrime). This was discussed [#mathlib4 > Placing a definition in `DedekindDomain.Ideal` @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Placing.20a.20definition.20in.20.60DedekindDomain.2EIdeal.60/near/511647129). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra
label:t-algebra$
11/1 Mathlib/RingTheory/DedekindDomain/Ideal.lean 1 5 ['Louddy', 'Ruben-VandeVelde', 'github-actions'] Ruben-VandeVelde
assignee:Ruben-VandeVelde
1
31-28220
1 month ago
56-29490
1 month ago
56-29544
56 days
21276 GabinKolly
author:GabinKolly
feat(ModelTheory/Substructures): define equivalences between equal substructures Define first-order equivalences between equal substructures, and prove related properties. --- This is some preparatory work for #18876 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-logic awaiting-author 62/0 Mathlib/ModelTheory/Substructures.lean 1 19 ['GabinKolly', 'YaelDillies', 'fpvandoorn', 'github-actions', 'grunweg'] nobody 1
31-11500
1 month ago
31-11500
1 month ago
46-55730
46 days
23955 Louddy
author:Louddy
feat: Ideal.count_associates_eq Add variant of `UniqueFactorizationMonoid.count_normalizedFactors_eq` for associated Ideals. This is convenient when you need to talk about an element as `a₀ = x ^ n * a`. Note the file is slightly over the 1500 lines limit, I hope that is ok. 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/) new-contributor t-algebra
label:t-algebra$
35/1 Mathlib/RingTheory/DedekindDomain/Ideal.lean 1 7 ['Louddy', 'Ruben-VandeVelde', 'alreadydone', 'github-actions', 'grunweg'] kbuzzard
assignee:kbuzzard
1
26-44624
26 days ago
26-44624
26 days ago
53-45384
53 days
23964 BoltonBailey
author:BoltonBailey
docs: Add documentation arbitrarily @mattrobball asked in the Mathlib Community meeting today what it would look like if we asked Claude code to give us improved documentation. I made this draft PR by selecting five declarations arbitrarily from `nolints.json` and asking Cursor to document them. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author documentation 52/14 Mathlib/Algebra/Homology/Homotopy.lean,Mathlib/Analysis/BoxIntegral/Partition/Filter.lean,Mathlib/Control/Monad/Cont.lean,Mathlib/Data/Stream/Defs.lean,Mathlib/LinearAlgebra/AffineSpace/AffineMap.lean 5 10 ['ADedecker', 'BoltonBailey', 'eric-wieser', 'github-actions', 'jcommelin', 'mattrobball'] nobody 1
25-49669
25 days ago
25-49669
25 days ago
33-13460
33 days
10235 urkud
author:urkud
feat: add `Decidable`, `Fintype`, `Encodable` linters This PR ports the `decidableClassical`, `fintypeFinite` and `encodableCountable` linters from mathlib3: all three are environment linters which flag declarations that have a hypothesis `[Decidable p]` etc., but do not use the underlying assumption in this type. Restructuring the code can make the statement more general. The implementation is in fact quite general, and can easily adapt to include further types. PRs #17518 and #17519 are two examples of further such linters. --- Please don't fix the failures related to `HasFDerivWithinAt.pi`. Finiteness assumptions in these lemmas will be completely removed during porting to TVS. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-bench large-import t-linter t-meta awaiting-author 123/4 Mathlib.lean,Mathlib/Computability/Halting.lean,Mathlib/Computability/TuringMachine.lean,Mathlib/Data/Fintype/Quotient.lean,Mathlib/Logic/Basic.lean,Mathlib/Logic/Encodable/Basic.lean,Mathlib/NumberTheory/JacobiSum/Basic.lean,Mathlib/Order/Heyting/Regular.lean,Mathlib/Tactic.lean,Mathlib/Tactic/GeneralizeProofs.lean,Mathlib/Tactic/Linter/UnusedAssumptionInType.lean 11 n/a ['Command-Master', 'github-actions', 'grunweg', 'kmill', 'leanprover-bot', 'urkud'] nobody 1
23-5887
23 days ago
unknown
unknown
21624 sinhp
author:sinhp
feat(CategoryTheory): The (closed) monoidal structure on the product category of families of (closed) monoidal categories Given a family of closed monoidal categories, we show that the product of these categories is a closed monoidal category with the pointwise monoidal structure. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory awaiting-author 144/0 Mathlib.lean,Mathlib/CategoryTheory/Pi/Basic.lean,Mathlib/CategoryTheory/Pi/Monoidal.lean,Mathlib/CategoryTheory/Pi/MonoidalClosed.lean 4 19 ['TwoFX', 'YaelDillies', 'b-mehta', 'github-actions', 'jcommelin', 'sinhp'] nobody 1
20-45417
20 days ago
20-45417
20 days ago
54-54882
54 days
22018 maddycrim
author:maddycrim
feat(RingTheory/Localization/Pi): localization of a finite direct product where each semiring in product has maximal nilradical is a projection For noncomputable def `surjectivePiNilradicalIsMaximal` : Let `M` be a submonoid of a direct product of commutative rings `R i`. If each `R i` has maximal nilradical then the direct product `∏ R i` surjects onto the localization of `∏ R i` at `M`. --- [![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$
28/0 Mathlib/RingTheory/Localization/Pi.lean 1 24 ['Paul-Lez', 'alreadydone', 'erdOne', 'github-actions', 'grunweg', 'jcommelin', 'maddycrim'] mariainesdff
assignee:mariainesdff
1
19-29279
19 days ago
64-12686
2 months ago
110-85911
110 days
23368 b-reinke
author:b-reinke
feat(GroupTheory/FreeGroup/ReducedWords): add theory of reduced words Upstreamed from the [EquationalTheories](https://github.com/teorth/equational_theories) project. This PR adds the file `GroupTheory/FreeGroup/ReducedWords.lean`, where the predicate of reduced words is defined. It is shown that `reduce` and `toWord` produce reduced words. This is done in preparation for the theory of cyclically reduced words. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-geometric-group-theory t-algebra
label:t-algebra$
104/0 Mathlib.lean,Mathlib/GroupTheory/FreeGroup/ReducedWords.lean 2 37 ['b-reinke', 'github-actions', 'tb65536', 'vlad902'] nobody 2
14-59970
14 days ago
74-25781
2 months ago
74-33611
74 days
25188 vlad902
author:vlad902
feat: add lemmas about `List.scanr` I add basic lemmas to reason about `List.scanr`, and slightly clean-up the file and add some basic lemmas to keep the API unified with the one for `List.scanl`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data 84/18 Mathlib/Data/List/Scan.lean 1 5 ['b-mehta', 'github-actions', 'vlad902'] nobody 1
14-48841
14 days ago
14-49069
14 days ago
14-72569
14 days
23684 alreadydone
author:alreadydone
feat(RingTheory): integral extensions of comm. rings are local homs --- The import increase only affects one file so I hope it's okay. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-algebra
label:t-algebra$
57/65 Mathlib/Algebra/Field/Equiv.lean,Mathlib/Algebra/Group/Invertible/Basic.lean,Mathlib/Algebra/GroupWithZero/Units/Basic.lean,Mathlib/AlgebraicGeometry/Morphisms/Proper.lean,Mathlib/FieldTheory/LinearDisjoint.lean,Mathlib/LinearAlgebra/Dimension/Localization.lean,Mathlib/RingTheory/Artinian/Ring.lean,Mathlib/RingTheory/IntegralClosure/Algebra/Defs.lean,Mathlib/RingTheory/IntegralClosure/IsIntegralClosure/Basic.lean,Mathlib/RingTheory/LinearDisjoint.lean,Mathlib/RingTheory/Localization/FractionRing.lean,Mathlib/RingTheory/Localization/Integral.lean,Mathlib/RingTheory/SimpleRing/Field.lean 13 4 ['alreadydone', 'github-actions', 'xroblot'] nobody 1
13-6805
13 days ago
65-72197
2 months ago
65-72217
65 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 7 ['Parcly-Taxel', 'YaelDillies', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant'] nobody 1
12-45087
12 days ago
12-45105
12 days ago
59-44919
59 days
22919 plp127
author:plp127
feat(Data/Fintype/Pi): Make `Fintype` instance for `RelHom`s computable Makes the `Fintype` instance for rel homs computable. See this [Zulip](https://leanprover.zulipchat.com/#narrow/channel/113489-new-members/topic/Classical.20vs.20constructive.20logic.20in.20computation/near/496220816) message. --- - [x] depends on: #24748 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data awaiting-author 178/44 Mathlib/Combinatorics/SimpleGraph/Basic.lean,Mathlib/Combinatorics/SimpleGraph/Coloring.lean,Mathlib/Combinatorics/SimpleGraph/Maps.lean,Mathlib/Data/Fintype/CardEmbedding.lean,Mathlib/Data/Fintype/Pi.lean 5 29 ['IvanRenison', 'b-mehta', 'eric-wieser', 'fpvandoorn', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'plp127'] b-mehta
assignee:b-mehta
1
11-58021
11 days ago
11-58021
11 days ago
73-73341
73 days
21950 erdOne
author:erdOne
feat(NumberTheory/Padics): the completion of `ℚ` at a finite place is `ℚ_[p]` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-number-theory 253/1 Mathlib.lean,Mathlib/Algebra/GroupWithZero/WithZero.lean,Mathlib/NumberTheory/Padics/HeightOneSpectrum.lean,Mathlib/NumberTheory/Padics/PadicNumbers.lean,Mathlib/Topology/Algebra/Valued/WithVal.lean,Mathlib/Topology/Algebra/WithZeroMulInt.lean,Mathlib/Topology/Algebra/WithZeroTopology.lean 7 22 ['Ruben-VandeVelde', 'erdOne', 'github-actions', 'leanprover-community-bot-assistant', 'pechersky', 'smmercuri', 'xroblot'] nobody 1
9-68894
9 days ago
9-68894
9 days ago
51-21490
51 days
25315 ocfnash
author:ocfnash
feat: add `simp` to lemma `Fin.coe_ofNat_eq_mod` One consequence is that `simp` can now prove things like this: ```lean example : (3 : Fin 10).val = 3 := by simp example : (4 : Fin 10).val = 4 := by simp example : (5 : Fin 10).val = 5 := by simp ``` previously this only this only worked up to `(2 : Fin 10).val = 2` (via lemmas like `Fin.val_two`). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data 32/28 Archive/Imo/Imo2024Q5.lean,Mathlib/AlgebraicTopology/DoldKan/Faces.lean,Mathlib/Analysis/CStarAlgebra/SpecialFunctions/PosPart.lean,Mathlib/Data/Fin/Basic.lean,Mathlib/Data/Fin/Parity.lean,Mathlib/Data/Fin/Rev.lean,Mathlib/GroupTheory/CommutingProbability.lean,Mathlib/GroupTheory/Perm/Fin.lean,Mathlib/RingTheory/ChainOfDivisors.lean,MathlibTest/matrix.lean 10 25 ['b-mehta', 'eric-wieser', 'github-actions', 'leanprover-bot', 'mattrobball', 'ocfnash'] nobody 1
9-18565
9 days ago
10-11743
10 days ago
10-11733
10 days
24777 joelriou
author:joelriou
feat(CategoryTheory): abstract argument for the stability under transfinite compositions If a class of morphisms is multiplicative, respects isomorphisms and is stable under filtered colimits, then it is stable under transfinite compositions. (This simplifies the proof in the case of monomorphisms in Grothendieck abelian categories, for isomorphisms, and in #23282, we shall apply this to monomorphisms in `Type`.) --- - [x] depends on: #24773 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-category-theory 122/116 Mathlib/CategoryTheory/Abelian/GrothendieckAxioms/Colim.lean,Mathlib/CategoryTheory/Abelian/GrothendieckCategory/EnoughInjectives.lean,Mathlib/CategoryTheory/Abelian/GrothendieckCategory/Monomorphisms.lean,Mathlib/CategoryTheory/MorphismProperty/Limits.lean,Mathlib/CategoryTheory/MorphismProperty/TransfiniteComposition.lean 5 12 ['callesonne', 'github-actions', 'joelriou', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody 1
8-11882
8 days ago
9-4698
9 days ago
21-28102
21 days
24514 b-mehta
author:b-mehta
chore(Int/GCD): use fuel in xgcd Modify the definition of xgcd to use fuel recursion, to allow it to be reduced in the kernel. As a consequence, this means the evaluation of field operations in ZMod p become provable by `rfl` and `decide`. Zulip discussion: https://leanprover.zulipchat.com/#narrow/channel/270676-lean4/topic/opaque.20recursion.20definitions.20break.20mergeSort.20decidability --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data 44/22 Mathlib/Data/Int/GCD.lean 1 4 ['b-mehta', 'eric-wieser', 'github-actions', 'nomeata', 'urkud'] nobody 1
7-84218
7 days ago
39-19437
1 month ago
39-19489
39 days
23970 AntoineChambert-Loir
author:AntoineChambert-Loir
feat(GroupTheory/GroupAction/SubMulAction/OfFixingSubgroup): action of the fixing Subgroup on the complement of a set Introduce the `SubMulAction` of a `fixingSubgroup` of a subset on the complement of that set. Develop relations between these and `SubMulAction` of stabilizers. --- - [x] depends on: #23386 - [x] depends on: #23962 - [x] depends on: #24107 - [x] depends on: #24117 - [x] depends on: #24167 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra delegated
label:t-algebra$
449/4 Mathlib.lean,Mathlib/Algebra/Group/End.lean,Mathlib/GroupTheory/GroupAction/FixingSubgroup.lean,Mathlib/GroupTheory/GroupAction/MultipleTransitivity.lean,Mathlib/GroupTheory/GroupAction/SubMulAction.lean,Mathlib/GroupTheory/GroupAction/SubMulAction/OfFixingSubgroup.lean 6 29 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib-bors', 'mathlib4-dependent-issues-bot', 'riccardobrasca'] riccardobrasca
assignee:riccardobrasca
1
6-35345
6 days ago
6-35345
6 days ago
13-15466
13 days
24480 mariainesdff
author:mariainesdff
feat(RingTheory/DividedPowers/SubPDIdeal): add SubDPIdeal Let `A` be a commutative (semi)ring and let `I` be an ideal of `A` with a divided power structure `hI`. A subideal `J` of `I` is a *sub-dp-ideal* of `(I, hI)` if, for all `n ∈ ℕ > 0` and all `x ∈ J`, `hI.dpow n x ∈ J`. The "TODOs" listed on the file docstring have been formalized by the authors and will be added in subsequent PRs. Co-authored-by: @AntoineChambert-Loir --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-number-theory ready-to-merge delegated
label:t-algebra$
373/0 Mathlib.lean,Mathlib/RingTheory/DividedPowers/SubDPIdeal.lean,Mathlib/RingTheory/Ideal/Span.lean 3 20 ['AntoineChambert-Loir', 'github-actions', 'mathlib-bors', 'riccardobrasca'] riccardobrasca
assignee:riccardobrasca
1
6-35277
6 days ago
6-36888
6 days ago
33-65896
33 days
25364 Paul-Lez
author:Paul-Lez
feat(Analysis/SpecialFunction/NthRoot): definition and basic API of Real.nthRoot Co-authored-by: Eric Wieser --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra WIP
label:t-algebra$
256/0 Mathlib/Analysis/SpecialFunctions/NthRoot.lean,Mathlib/Data/Sign.lean 2 16 ['eric-wieser', 'fpvandoorn', 'github-actions', 'j-loreaux', 'madvorak'] nobody 1
5-35397
5 days ago
7-23524
7 days ago
0-42
42 seconds
25139 kckennylau
author:kckennylau
feat(RingTheory): basis for `Polynomial.degreeLT` Linear algebra results about the module `R[x]_n` of polynomials with degree `< n`. Co-authored-by: Anne Baanen --- - [x] depends on: #25270 Used in a future resultant PR from branch [kckennylau/resultant](https://github.com/leanprover-community/mathlib4/tree/kckennylau/resultant). This file is split from that branch because there are already over 1000 lines of code. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra awaiting-author
label:t-algebra$
195/2 Mathlib.lean,Mathlib/Algebra/Polynomial/Taylor.lean,Mathlib/RingTheory/Polynomial/DegreeLT.lean 3 108 ['YaelDillies', 'erdOne', 'github-actions', 'kbuzzard', 'kckennylau', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody 1
5-9619
5 days ago
5-43801
5 days ago
4-17234
4 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'] nobody 1
4-68137
4 days ago
5-6071
5 days ago
6-16421
6 days
11968 JovanGerb
author:JovanGerb
feat: improvements to RefinedDiscrTree This PR defines `RefinedDiscrTree`, which is an improved version of `DiscrTree` with many new features, such as - indexing lambda terms, dependent forall terms, and bound variables. - giving a score to matches, in order to sort them - indexing star patterns so that `a+b` and `a+a` are indexed differently - taking into account eta reductions, so that `exp` can still be matched with the library pattern `fun x => exp (f x)`. This PR makes `RefinedDiscrTree` into a lazy data structure, meaning that it can be used without a cache, just like `LazyDiscrTree`. This PR also removes these features: - indexing `fun x => x` as `id` - indexing `fun x => f x + g x` as `f + g`, and similarly for `-`, `*`, `/`, `⁻¹`, `^`. - indexing `fun _ => 42` as `42` These equivalent indexings do not hold definitionally in the `reducible` transparency, which is the transparency that is used for unification when using a discrimination tree. Therefore, indexing these different expressions the same is actually inefficient rather than helpful. This is part of the bigger #11768, which uses this discrimination tree for a library rewriting tactic. This replaces an older version of `RefinedDiscrTree`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) file-removed new-contributor t-meta 1631/1242 Mathlib.lean,Mathlib/Lean/Meta/RefinedDiscrTree.lean,Mathlib/Lean/Meta/RefinedDiscrTree/Basic.lean,Mathlib/Lean/Meta/RefinedDiscrTree/Encode.lean,Mathlib/Lean/Meta/RefinedDiscrTree/Initialize.lean,Mathlib/Lean/Meta/RefinedDiscrTree/Lookup.lean,Mathlib/Lean/Meta/RefinedDiscrTree/Pi.lean,Mathlib/Tactic.lean,Mathlib/Tactic/FunProp.lean,Mathlib/Tactic/FunProp/Elab.lean,Mathlib/Tactic/FunProp/StateList.lean,Mathlib/Tactic/FunProp/Theorems.lean,Mathlib/Tactic/FunProp/Types.lean,Mathlib/Topology/Defs/Basic.lean,MathlibTest/RefinedDiscrTree.lean,scripts/noshake.json 16 79 ['0art0', 'JovanGerb', 'eric-wieser', 'github-actions', 'grunweg', 'joneugster', 'leanprover-bot', 'leanprover-community-bot-assistant', 'rosborn'] nobody 1
4-35094
4 days ago
4-85032
4 days ago
237-83175
237 days
24465 adomani
author:adomani
feat: a linter to enforce formatting This linter enforces that the hypotheses of every declaration are correctly formatted. This already required multiple PRs to make mathlib compliant. Ideally, little by little the linter can be extended to format more of mathlib. --- The default linter option is `false`, but the lakefile enforces it to be `true`. This means that the linter does not run on `MathlibTest`. However, the tests should still be compliant, since the default option was `true` in development and the tests were fixed. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-linter maintainer-merge 876/4 Mathlib.lean,Mathlib/Algebra/Group/Int/Defs.lean,Mathlib/Algebra/Group/Nat/Defs.lean,Mathlib/Algebra/Ring/Int/Defs.lean,Mathlib/Data/FunLike/Basic.lean,Mathlib/Data/SetLike/Basic.lean,Mathlib/Init.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter/CommandStart.lean,Mathlib/Tactic/Simps/NotationClass.lean,MathlibTest/CommandStart.lean,MathlibTest/EuclideanSpace.lean,MathlibTest/Simps.lean,MathlibTest/Traversable.lean,MathlibTest/antidiagonal.lean,MathlibTest/delabLinearIndependent.lean,MathlibTest/matrix.lean,MathlibTest/norm_num.lean,MathlibTest/set_like.lean,MathlibTest/vec_notation.lean 20 89 ['Parcly-Taxel', 'adomani', 'eric-wieser', 'github-actions', 'grunweg', 'leanprover-community-bot-assistant'] grunweg
assignee:grunweg
1
4-30689
4 days ago
27-42382
27 days ago*
40-47103
40 days*
25482 grunweg
author:grunweg
chore(aesop_cat): update comment Since mathlib includes leanprover/lean4#7448, update the comment accordingly. #25475 shows that this fast-path is still beneficial: so leave it, but update its comment accordingly. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory 4/4 Mathlib/CategoryTheory/Category/Basic.lean 1 2 ['JovanGerb', 'github-actions', 'grunweg'] nobody 1
4-24173
4 days ago
4-26873
4 days ago
4-26925
4 days
25265 FMLJohn
author:FMLJohn
feat(Order/SupClosed): `compl_image_latticeClosure` and `compl_image_latticeClosure_eq_of_compl_image_eq_self` The main results in this pull request are: 1. `compl_image_latticeClosure`: given any Boolean algebra `α` and `s : Set α`, `compl '' latticeClosure s` is the same as `latticeClosure (compl '' s)`; 2. `compl_image_latticeClosure_eq_of_compl_image_eq_self`: given any Boolean algebra `α` and `s : Set α` such that `compl '' s = s`, we have `compl '' latticeClosure s = latticeClosure s`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) maintainer-merge t-order 59/1 Mathlib/Order/SupClosed.lean 1 8 ['FMLJohn', 'YaelDillies', 'github-actions'] bryangingechen
assignee:bryangingechen
1
4-22149
4 days ago
7-2121
7 days ago
11-11741
11 days
25369 Paul-Lez
author:Paul-Lez
feat(Order/Fin/CircularOrder): add some basic results about the circular order on Fin Co-authored-by: Oliver Nash --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order awaiting-author 33/0 Mathlib.lean,Mathlib/Order/Circular.lean,Mathlib/Order/Fin/CircularOrder.lean 3 11 ['Paul-Lez', 'YaelDillies', 'eric-wieser', 'github-actions'] bryangingechen
assignee:bryangingechen
1
4-22121
4 days ago
4-22121
4 days ago
2-19068
2 days
25172 eric-wieser
author:eric-wieser
feat: restricting `Affine.Simplex` to an affine subspace that contains it Also removes a redundant `Nonempty` argument. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) maintainer-merge t-euclidean-geometry 68/5 Mathlib/LinearAlgebra/AffineSpace/AffineSubspace/Basic.lean,Mathlib/LinearAlgebra/AffineSpace/Independent.lean 2 10 ['eric-wieser', 'github-actions', 'jsm28', 'ocfnash'] nobody 1
4-16192
4 days ago
15-26171
15 days ago
15-67045
15 days
25255 Raph-DG
author:Raph-DG
feat(RingTheory): Order of vanishing in a ring In this PR we define the order of vanishing of a ring and its extension to elements of the function field (as in stacks project 02MD) as well as some basic API. Note that I'm slightly unsure that some of the lemmas used to prove this are at the right level of generality, and further I'm not quite sure where some of these lemmas belong (as indicated by the comments in the main OrderOfVanishing.lean file). Any comments about this would be very much appreciated. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) maintainer-merge new-contributor t-algebra RFC
label:t-algebra$
247/0 Mathlib.lean,Mathlib/Algebra/Order/Monoid/Unbundled/WithTop.lean,Mathlib/RingTheory/Artinian/Module.lean,Mathlib/RingTheory/Ideal/Operations.lean,Mathlib/RingTheory/Ideal/Quotient/Operations.lean,Mathlib/RingTheory/OrderOfVanishing.lean 6 83 ['Raph-DG', 'chrisflav', 'erdOne', 'github-actions', 'jcommelin'] nobody 1
3-81423
3 days ago
3-82009
3 days ago
10-61393
10 days
23669 erdOne
author:erdOne
feat(FieldTheory): abelian extensions --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra awaiting-author
label:t-algebra$
74/0 Mathlib.lean,Mathlib/FieldTheory/Galois/Abelian.lean,Mathlib/NumberTheory/Cyclotomic/Gal.lean 3 6 ['acmepjz', 'alreadydone', 'chrisflav', 'erdOne', 'github-actions', 'xroblot'] nobody 2
3-50620
3 days ago
36-34663
1 month ago
29-68817
29 days
21265 ADedecker
author:ADedecker
feat: some lemmas about pointwise actions of units on filters and uniformities --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-topology delegated
label:t-algebra$
45/0 Mathlib/Order/Filter/Pointwise.lean,Mathlib/Topology/Algebra/UniformMulAction.lean 2 8 ['github-actions', 'grunweg', 'mathlib-bors', 'ocfnash'] nobody 1
3-43644
3 days ago
114-83977
3 months ago
15-25642
15 days
22366 kim-em
author:kim-em
feat: `check_equalities` tactic for diagnosing defeq problems The `check_equalities` tactic, which checks the typing of equalities in the goal, reporting discrepancies between the implicit type argument of the equality, and the inferred types of the left and right hand sides, at "instances and reducible" transparency. Reports from this tactic do not necessarily indicate a problem, although typically `simp` should reduce rather than increase the reported discrepancies. `check_equalities` may be useful in diagnosing uses of `erw`. t-meta delegated 119/3 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Basic.lean,Mathlib/Tactic/CategoryTheory/CheckCompositions.lean,Mathlib/Tactic/CheckEqualities.lean,Mathlib/Tactic/Common.lean,MathlibTest/check_equalities.lean 7 13 ['adomani', 'b-mehta', 'eric-wieser', 'github-actions', 'grunweg', 'mathlib-bors'] nobody 1
3-43553
3 days ago
87-17765
2 months ago
15-14325
15 days
18693 Ruben-VandeVelde
author:Ruben-VandeVelde
feat: add ConjRootClass Co-authored-by: FR --- From #6718 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra delegated
label:t-algebra$
213/0 Mathlib.lean,Mathlib/FieldTheory/Minpoly/ConjRootClass.lean,Mathlib/FieldTheory/Minpoly/IsConjRoot.lean 3 16 ['LessnessRandomness', 'Vierkantor', 'alreadydone', 'github-actions', 'grunweg', 'mathlib-bors'] Vierkantor
assignee:Vierkantor
2
3-43512
3 days ago
14-19065
14 days ago
94-8480
94 days
23240 urkud
author:urkud
feat(Topology/Maps): `IsOpenMap` and `ClusterPt` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology delegated 17/4 Mathlib/Topology/Maps/Basic.lean 1 8 ['eric-wieser', 'github-actions', 'grunweg', 'mathlib-bors', 'urkud'] nobody 1
3-20874
3 days ago
77-76255
2 months ago
0-12104
3 hours
25059 s235282
author:s235282
feat(Combinatorics/SimpleGraph/Bipartite): a graph is 2-colorable iff it's bipartite Define a predicate for a simple graph to be bipartite (`def IsBipartite (G : SimpleGraph V) : Prop := G.Colorable 2`) and prove ` G.IsBipartite ↔ ∃ s t : Set V, G.IsBipartiteWith s t`. --- This is my first attempt at contributing to mathlib and therefore I have a couple of points of uncertainty related to: - Naming conventions for theorems - Seeing a lot of isBipartite vs IsBipartite in the original work. What do we want to go with when? - Definition placement - Where should I put the IsBipartite definition. - Structure of biimplication theorems - Should I combine the different lemmas into 1 bgi theorem? Feedback is greatly appreciated :) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import maintainer-merge new-contributor t-combinatorics 36/3 Mathlib/Combinatorics/SimpleGraph/Bipartite.lean 1 30 ['YaelDillies', 'github-actions', 'mitchell-horner', 's235282'] nobody 2
2-36455
2 days ago
2-37002
2 days ago
8-84432
8 days
24261 Paul-Lez
author:Paul-Lez
chore: replace `WithLp.equiv` with a new pair `WithLp.toLp`/`WithLp.ofLp` This PR does the following: - deprecate `WithLp.equiv` - Add `WithLp.toLp` and `WithLp.ofLp` (for consistency with other equivalences to type synonyms) See [Zulip discussion](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/defeq.20abuse.20in.20.60WithLp.60) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis 759/366 Mathlib/Algebra/Module/ZLattice/Covolume.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/Matrix.lean,Mathlib/Analysis/Normed/Algebra/UnitizationL1.lean,Mathlib/Analysis/Normed/Lp/PiLp.lean,Mathlib/Analysis/Normed/Lp/ProdLp.lean,Mathlib/Analysis/Normed/Lp/WithLp.lean,Mathlib/Analysis/Quaternion.lean,Mathlib/Analysis/RCLike/Inner.lean,Mathlib/Analysis/SpecialFunctions/Gaussian/FourierTransform.lean,Mathlib/Combinatorics/Additive/AP/Three/Behrend.lean,Mathlib/Geometry/Euclidean/Angle/Unoriented/CrossProduct.lean,Mathlib/LinearAlgebra/Matrix/Hermitian.lean,Mathlib/LinearAlgebra/Matrix/LDL.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,MathlibTest/EuclideanSpace.lean 24 50 ['Paul-Lez', 'YaelDillies', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant'] nobody 1
2-35204
2 days ago
2-35224
2 days ago
33-31560
33 days
24661 edegeltje
author:edegeltje
feat(Tactic/Algebraize): Allow the `algebraize` tactic to use lemmas which don't (directly) mention RingHom This PR allows the `algebraize` tactic to be applied in more cases. Specifically, in cases where the assumption is not (directly) about RingHom, it should still be able to apply lemmas. Written at the suggestion of @chrisflav , with the following example usecase: ```lean-4 import Mathlib open AlgebraicGeometry attribute [algebraize flat_of_flat] Flat -- pretend this is added where `AlgebraicGeometry.Flat` is defined lemma flat_of_flat {R S : Type u} [CommRing R] [CommRing S] (f : R →+* S) (h : Flat (Spec.map (CommRingCat.ofHom f))) : @Module.Flat R S _ _ f.toAlgebra.toModule := by have : f.Flat := sorry -- supposedly, this is true. ask christian. algebraize [f] assumption set_option tactic.hygienic false -- allow the tactic to produce accessible names for testing example {R S : Type u} [CommRing R] [CommRing S] (f : R →+* S) (h : Flat (Spec.map (CommRingCat.ofHom f))) : True := by algebraize [f] guard_hyp algebraizeInst : Module.Flat R S -- used to fail, succeeds now trivial ``` the key changes that makes this possible are the following: - a different way of making lemma/type applications, creating a term which can be added to the context - a different way of checking that the previously mentioned term actually relevant w/r/t the arguments provided to the tactic The previous check was ad-hoc and flimsy, making requirements of the precise order and the types of the arguments of lemmas or definitions, which resulted in the lemma being applicable in limited cases only. Now we still have some requirements, but these are less stringent. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta awaiting-author enhancement 147/62 Mathlib/Tactic/Algebraize.lean,MathlibTest/algebraize.lean 2 34 ['callesonne', 'chrisflav', 'edegeltje', 'github-actions'] nobody 1
2-35124
2 days ago
2-35124
2 days ago
26-65389
26 days
25094 grunweg
author:grunweg
feat(Tactic/Positivity): extend EReal support for numeric casts Extend `pos_of_isNat` and `nonneg_of_isNat` to cover monoids which are not necessarily semirings, like EReal. [Zulip discussion](https://leanprover.zulipchat.com/#narrow/channel/113488-general/topic/.22Missing.20Tactics.22.20list/near/519660424) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta awaiting-author 70/36 Mathlib/Tactic/Positivity/Core.lean,MathlibTest/positivity.lean 2 19 ['Paul-Lez', 'YaelDillies', 'github-actions', 'grunweg', 'leanprover-bot', 'leanprover-community-bot-assistant', 'leanprover-community-mathlib4-bot'] nobody 1
2-34924
2 days ago
2-34924
2 days ago
13-6021
13 days
25089 Bergschaf
author:Bergschaf
feat(Order/Sublocale): definition of sublocales There are several possible definition of sublocales. I used one from [nlab](https://ncatlab.org/nlab/show/sublocale) which states that a sublocale is a subset of a locale which is closed under all meets and for any ∈ S and x ∈ X, we have x ⇨ s ∈ S. This PR also includes an order isomorphism between (Nucleus)ᵒᵈ and Sublocale. --- I am open to better name suggestions for the order isomorphism. - [x] depends on: #24941 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) maintainer-merge t-order 265/8 Mathlib.lean,Mathlib/Order/Hom/Lattice.lean,Mathlib/Order/Nucleus.lean,Mathlib/Order/Sublocale.lean,Mathlib/Order/Synonym.lean,docs/references.bib 6 71 ['Bergschaf', 'YaelDillies', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'xhalo32'] nobody 1
2-955
2 days ago
2-955
2 days ago
15-66778
15 days
25501 eric-wieser
author:eric-wieser
fix: eliminate metadata in linarith Otherwise this interferes with the `answer()` elaborator from formal-conjectures. Diagnosed using #25500. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta delegated bug 7/1 Mathlib/Tactic/Linarith/Parsing.lean,MathlibTest/linarith.lean 2 8 ['adomani', 'b-mehta', 'github-actions', 'j-loreaux', 'leanprover-bot', 'mathlib-bors'] nobody 1
1-85708
1 day ago
2-1462
2 days ago
1-78612
1 day
20924 tomaz1502
author:tomaz1502
feat(Computability/QueryComplexity): Oracle-based computation This PR adds the types and lemmas for oracle-based computation. In this model, computations are run on a monad which also counts the number of oracle queries executed. With it, it becomes possible to reason about the upper bound of the query complexity of algorithms. In the future, we could extend this work to include the necessary bits from information theory and probability to also reason about lower bounds on query complexity, like the work in https://github.com/girving/debate. Zulip discussion: https://leanprover.zulipchat.com/#narrow/channel/144837-PR-reviews/topic/.2318629.20runtime.20complexity.20of.20sorting.20a.20list Co-authored-by: Geoffrey Irving --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-computability 305/0 Mathlib.lean,Mathlib/Computability/QueryComplexity/Basic.lean,Mathlib/Computability/QueryComplexity/Defs.lean 3 58 ['eric-wieser', 'girving', 'github-actions', 'quangvdao', 'tomaz1502'] nobody 1
1-15090
1 day ago
138-13504
4 months ago
138-13495
138 days
24382 joelriou
author:joelriou
feat(CategoryTheory): pseudofunctors from strict bicategories This PR provides an API for pseudofunctors `F` from a strict bicategory `B`. In particular, this shall apply to pseudofunctors from locally discrete bicategories. We first introduce more flexible variants of `mapId` and `mapComp`: for example, if `f` and `g` are composable morphisms and `fg` is such that `h : fg = f ≫ f`, we provide an isomorphism `F.mapComp' f g fg h : F.map fg ≅ F.map f ≫ F.map g`. We study the compatibilities of these isomorphisms with respect to composition with identities and associativity. Secondly, given a commutative square `t ≫ r = l ≫ b` in `B`, we construct an isomorphism `F.map t ≫ F.map r ≅ F.map l ≫ F.map b`. Co-authored-by: Christian Merten --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) maintainer-merge t-category-theory 168/0 Mathlib.lean,Mathlib/CategoryTheory/Bicategory/Functor/Pseudofunctor.lean,Mathlib/CategoryTheory/Bicategory/Functor/Strict.lean 3 17 ['callesonne', 'erdOne', 'github-actions', 'joelriou'] nobody 1
1-12557
1 day ago
1-78341
1 day ago
44-5911
44 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$
92/1 Mathlib.lean,Mathlib/Algebra/Ring/Equiv.lean,Mathlib/RingTheory/RingHom/FaithfullyFlat.lean,Mathlib/RingTheory/RingHom/Flat.lean 4 4 ['chrisflav', 'erdOne', 'github-actions', 'mathlib4-dependent-issues-bot'] nobody 1
0-42212
11 hours ago
30-36220
30 days ago
30-37286
30 days
25050 linesthatinterlace
author:linesthatinterlace
feat: Add `Vector`/`List.Vector` equivalence Adds an equivalence between `Vector` and `List.Vector`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data 125/17 Mathlib/Data/Vector/Basic.lean,Mathlib/Data/Vector/Defs.lean,Mathlib/Logic/Equiv/Array.lean 3 57 ['digama0', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'linesthatinterlace'] nobody 1
0-37494
10 hours ago
0-40379
11 hours ago
6-55239
6 days
12934 grunweg
author:grunweg
chore: replace more uses of > or ≥ by < or ≤ These were flagged by the linter in https://github.com/leanprover-community/mathlib4/pull/12879: it is easy to simple avoid > or ≥ in hypotheses or haves. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author help-wanted 41/42 Archive/Imo/Imo1962Q1.lean,Archive/Imo/Imo1988Q6.lean,Archive/Imo/Imo1994Q1.lean,Archive/Imo/Imo2005Q3.lean,Archive/Imo/Imo2006Q3.lean,Archive/Imo/Imo2008Q2.lean,Archive/Imo/Imo2008Q3.lean,Archive/Imo/Imo2019Q4.lean,Archive/Sensitivity.lean,Archive/Wiedijk100Theorems/CubingACube.lean,Mathlib/Tactic/Linarith/Datatypes.lean,test/cancel_denoms.lean,test/congr.lean,test/interval_cases.lean,test/observe.lean 15 11 ['YaelDillies', 'adomani', 'github-actions', 'grunweg', 'jcommelin', 'urkud'] nobody 1
313-42770
10 months ago
326-52367
10 months ago
1-73101
1 day
12608 eric-wieser
author:eric-wieser
feat: allow `nsmul` / `zsmul` to be omitted again, with a warning --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-meta merge-conflict awaiting-author
label:t-algebra$
118/2 Mathlib.lean,Mathlib/Algebra/Group/Defs.lean,Mathlib/Tactic.lean,Mathlib/Tactic/DefaultFieldLinter.lean,scripts/noshake.json,test/default_field_linter.lean 6 12 ['YaelDillies', 'eric-wieser', 'fpvandoorn', 'github-actions'] nobody 1
313-42770
10 months ago
362-37834
11 months ago
5-72414
5 days
8519 eric-wieser
author:eric-wieser
refactor(LinearAlgebra/TensorProduct): golf using `liftAddHom` This new `TensorProduct.liftAddHom` doesn't require bilinearity, only that scalar multiplication can be moved between the arguments. While in theory we only need the `AddMonoidHom` version as it offers exactly the same generality, we first provide an unbundled `liftFun` as this seems to give a sizeable performance boost if used in downstream `lift` variants. --- - [x] depends on: #8571 - [x] depends on: #8584 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict awaiting-author
label:t-algebra$
53/50 Mathlib/Algebra/Category/AlgebraCat/Monoidal.lean,Mathlib/LinearAlgebra/TensorProduct.lean,Mathlib/LinearAlgebra/TensorProduct/Tower.lean 3 28 ['bustercopley', 'eric-wieser', 'jcommelin', 'jjaassoonn', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'mathlib-bors'] nobody 1
313-42767
10 months ago
462-15082
1 year ago
5-6524
5 days
9146 laughinggas
author:laughinggas
feat(Data/ZMod/Defs): Topological structure on `ZMod` Added a discrete topology structure to `ZMod n` for all `n` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-topology merge-conflict awaiting-author
label:t-algebra$
55/3 Mathlib.lean,Mathlib/Topology/Algebra/Constructions.lean,Mathlib/Topology/Algebra/Group/Basic.lean,Mathlib/Topology/Instances/ZMod.lean,Mathlib/Topology/Maps.lean 5 61 ['YaelDillies', 'eric-wieser', 'github-actions', 'jcommelin', 'laughinggas', 'mo271', 'urkud'] nobody 1
313-42767
10 months ago
494-50895
1 year ago
7-6153
7 days
6777 adomani
author:adomani
chore(Co*variantClass): replace eta-expanded (· * ·), (· + ·), (· ≤ ·), (· < ·) Replace `CovariantClass X X (· * ·) (· ≤ ·)` with -> `CovariantClass X X HMul.hMul LE.le` and similarly for `HAdd`, `LT`, `Contravariant`. This PR is inspired by [Issue #6646](https://github.com/leanprover-community/mathlib4/issues/6646) and, more specifically, [this comment](https://github.com/leanprover-community/mathlib4/issues/6646#issuecomment-1692792066). Note that https://github.com/leanprover/lean4/pull/2267 would make this unnecessary --- ```bash # First sed command: # the first captured pattern is `Co*variantClass ` # the second captured pattern is `` # the third captured pattern is `+` or `*` # the fourth captured pattern is `<` or `≤` # a match for `Co*variantClass ·) (· ·)` becomes # `Co*variantClass replaceop replaceop` # Second sed command: similar to the first, but looks for `(Function.swap (· ·))` sed -i ' s=\(Co[ntra]*variantClass \(..*\) \2 \)(· *\([+*]\) *·) (· *\([<≤]\) *·)=\1replaceop\3 replaceop\4=g s=\(Co[ntra]*variantClass \(..*\) \2 \)(\([Functio\.swap ]*\)(· *\([+*]\) *·)) (· *\([<≤]\) *·)=\1(\3replaceop\4) replaceop\5=g s=replaceop+=HAdd.hAdd=g s=replaceop\*=HMul.hMul=g s=replaceop<=LT.lt=g s=replaceop≤=LE.le=g s=\(Co[ntra]*variantClass N N\) (· \* ·) r=\1 HMul.hMul r=g s=\(Co[ntra]*variantClass N N (swap μ)\) (· ≤ ·)=\1 LE.le=g s=\(Co[ntra]*variantClass N N\) (swap (· \* ·)) r=\1 (swap HMul.hMul) r=g s=\(CovariantClass (Filter α) (Filter α)\) (· / ·) (· ≤ ·)=\1 HDiv.hDiv LE.le=g s=\(CovariantClass (Filter α) (Filter α)\) (swap (· / ·)) (· ≤ ·)=\1 (swap HDiv.hDiv) LE.le=g s=\(Co[ntra]*variantClass .* (fun x y .> . \* .)\) (· ≤ ·)=\1 LE.le=g s=\(Co[ntra]*variantClass .* (fun x y .> . \* .)\) (· < ·)=\1 LT.lt=g s=\(Co[ntra]*variantClass [^}]*\) (· ≤ ·)=\1 LE.le=g s=\(CovariantClass .* (Filter β)\) (· • ·) LE.le=\1 HSMul.hSMul LE.le=g ' $(git ls-files '*.lean') ``` [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict 703/678 Counterexamples/ZeroDivisorsInAddMonoidAlgebras.lean,Mathlib/Algebra/BigOperators/Basic.lean,Mathlib/Algebra/Bounds.lean,Mathlib/Algebra/CovariantAndContravariant.lean,Mathlib/Algebra/DirectSum/Internal.lean,Mathlib/Algebra/Group/UniqueProds.lean,Mathlib/Algebra/GroupPower/Order.lean,Mathlib/Algebra/MonoidAlgebra/Degree.lean,Mathlib/Algebra/Order/Archimedean.lean,Mathlib/Algebra/Order/Group/Abs.lean,Mathlib/Algebra/Order/Group/Defs.lean,Mathlib/Algebra/Order/Group/DenselyOrdered.lean,Mathlib/Algebra/Order/Group/MinMax.lean,Mathlib/Algebra/Order/Group/OrderIso.lean,Mathlib/Algebra/Order/Hom/Monoid.lean,Mathlib/Algebra/Order/Interval.lean,Mathlib/Algebra/Order/Kleene.lean,Mathlib/Algebra/Order/LatticeGroup.lean,Mathlib/Algebra/Order/Module.lean,Mathlib/Algebra/Order/Monoid/Basic.lean,Mathlib/Algebra/Order/Monoid/Cancel/Defs.lean,Mathlib/Algebra/Order/Monoid/Canonical/Defs.lean,Mathlib/Algebra/Order/Monoid/Defs.lean,Mathlib/Algebra/Order/Monoid/Lemmas.lean,Mathlib/Algebra/Order/Monoid/MinMax.lean,Mathlib/Algebra/Order/Monoid/NatCast.lean,Mathlib/Algebra/Order/Monoid/OrderDual.lean,Mathlib/Algebra/Order/Monoid/Prod.lean,Mathlib/Algebra/Order/Monoid/WithTop.lean,Mathlib/Algebra/Order/Monoid/WithZero/Basic.lean,Mathlib/Algebra/Order/Monoid/WithZero/Defs.lean,Mathlib/Algebra/Order/Nonneg/Ring.lean,Mathlib/Algebra/Order/Pointwise.lean,Mathlib/Algebra/Order/Positive/Ring.lean,Mathlib/Algebra/Order/Ring/Canonical.lean,Mathlib/Algebra/Order/Ring/Defs.lean,Mathlib/Algebra/Order/Ring/Lemmas.lean,Mathlib/Algebra/Order/Sub/Basic.lean,Mathlib/Algebra/Order/Sub/Canonical.lean,Mathlib/Algebra/Order/Sub/Defs.lean,Mathlib/Algebra/Order/WithZero.lean,Mathlib/Algebra/Parity.lean,Mathlib/Algebra/Star/Order.lean,Mathlib/Algebra/Tropical/Basic.lean,Mathlib/Analysis/Normed/Order/Lattice.lean,Mathlib/Data/DFinsupp/Lex.lean,Mathlib/Data/DFinsupp/Order.lean,Mathlib/Data/Finset/Fold.lean,Mathlib/Data/Finsupp/Lex.lean,Mathlib/Data/Finsupp/Order.lean,Mathlib/Data/List/BigOperators/Basic.lean,Mathlib/Data/List/BigOperators/Lemmas.lean,Mathlib/Data/Multiset/Basic.lean,Mathlib/Data/Nat/Cast/Order.lean,Mathlib/Data/PNat/Basic.lean,Mathlib/Data/Real/ENNReal.lean,Mathlib/Data/Real/NNReal.lean,Mathlib/Data/Set/Semiring.lean,Mathlib/Data/Sign.lean,Mathlib/MeasureTheory/Function/LpOrder.lean,Mathlib/MeasureTheory/Function/SimpleFuncDenseLp.lean,Mathlib/MeasureTheory/Measure/MeasureSpace.lean,Mathlib/MeasureTheory/Measure/VectorMeasure.lean,Mathlib/Order/ConditionallyCompleteLattice/Group.lean,Mathlib/Order/Filter/Basic.lean,Mathlib/Order/Filter/Pointwise.lean,Mathlib/Probability/Martingale/Basic.lean,Mathlib/Probability/Process/Stopping.lean,Mathlib/RingTheory/GradedAlgebra/Basic.lean,Mathlib/SetTheory/Cardinal/Basic.lean,Mathlib/SetTheory/Game/Basic.lean,Mathlib/SetTheory/Game/PGame.lean,Mathlib/SetTheory/Ordinal/Arithmetic.lean,Mathlib/SetTheory/Ordinal/Basic.lean,Mathlib/SetTheory/Ordinal/NaturalOps.lean,Mathlib/Tactic/GCongr/Core.lean,Mathlib/Tactic/Positivity/Basic.lean,Mathlib/Topology/ContinuousFunction/Algebra.lean,lean-toolchain,test/Recall.lean,test/propose.lean 81 36 ['adomani', 'alreadydone', 'digama0', 'eric-wieser', 'ericrbg', 'jcommelin', 'leanprover-bot', 'sgouezel'] nobody 1
313-42766
10 months ago
335-23470
11 months ago
35-56459
35 days
6403 FR-vdash-bot
author:FR-vdash-bot
chore: change instance priorities of `Ordered*` hierarchy --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) slow-typeclass-synthesis t-order t-algebra merge-conflict awaiting-author
label:t-algebra$
253/79 Mathlib/Algebra/Order/CompleteField.lean,Mathlib/Algebra/Order/Field/Canonical/Defs.lean,Mathlib/Algebra/Order/Field/Defs.lean,Mathlib/Algebra/Order/Group/Defs.lean,Mathlib/Algebra/Order/Monoid/Basic.lean,Mathlib/Algebra/Order/Monoid/Canonical/Defs.lean,Mathlib/Algebra/Order/Monoid/Defs.lean,Mathlib/Algebra/Order/Monoid/WithZero/Defs.lean,Mathlib/Algebra/Order/Ring/Canonical.lean,Mathlib/Algebra/Order/Ring/Defs.lean,Mathlib/Algebra/Order/Ring/Star.lean,Mathlib/Algebra/Order/WithZero.lean,Mathlib/Analysis/InnerProductSpace/Orientation.lean,Mathlib/LinearAlgebra/Orientation.lean,Mathlib/RingTheory/HahnSeries.lean,Mathlib/RingTheory/LaurentSeries.lean,Mathlib/Tactic/Positivity/Core.lean,Mathlib/Topology/Algebra/WithZeroTopology.lean 18 39 ['FR-vdash-bot', 'Vierkantor', 'digama0', 'eric-wieser', 'j-loreaux', 'leanprover-bot'] nobody 1
313-42765
10 months ago
371-86235
1 year ago
13-18399
13 days
3757 thorimur
author:thorimur
feat: config options for `fail_if_no_progress` This PR creates config options for `fail_if_no_progress` that allow the user to tweak what exactly counts as "progress". This includes whether to use defeq or `BEq`, what transparency to use, and which parts of the goal and local context to check. It also splits off the comparison functionality into `Mathlib.Lean.Meta.Compare`, which provides fully configurable comparison functions for common complex metaprogramming types not specific to `fail_if_no_progress`. These types are `Expr`, `LocalDecl`, `LocalContext`, `MetavarDecl`, `MVarId`, and `List MVarId`. --- See [zulip](https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/progress.20on.20fail_if_no_progress) for a couple review questions. Status update: this PR is now basically done, save for some extra tests which should probably be included. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta merge-conflict WIP 603/54 Mathlib.lean,Mathlib/Lean/Meta.lean,Mathlib/Lean/Meta/Compare.lean,Mathlib/Tactic/FailIfNoProgress.lean,test/fail_if_no_progress.lean 5 38 ['alexjbest', 'github-actions', 'joneugster', 'kim-em', 'thorimur'] nobody 1
313-42764
10 months ago
565-53950
1 year ago
45-49113
45 days
12751 Command-Master
author:Command-Master
feat: add lemmas for Nat/Bits, Nat/Bitwise and Nat/Size Remove `@[simp]` from `Nat.bit_false` and `Nat.bit_true`, as `bit0` and `bit1` are deprecated, and add some lemmas to `Bits`, `Bitwise` and `Size`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data new-contributor merge-conflict 66/7 Mathlib/Data/Nat/Bits.lean,Mathlib/Data/Nat/Bitwise.lean,Mathlib/Data/Nat/Multiplicity.lean,Mathlib/Data/Nat/Size.lean 4 26 ['Command-Master', 'Rida-Hamadani', 'Ruben-VandeVelde', 'YaelDillies', 'github-actions', 'jcommelin'] nobody 1
294-20067
9 months ago
299-36309
9 months ago
54-52408
54 days
15448 urkud
author:urkud
chore(*): deprecate `Option.elim'` Use `Option.elim` instead. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) tech debt merge-conflict awaiting-author 54/50 Mathlib/Algebra/BigOperators/Option.lean,Mathlib/Algebra/MvPolynomial/Equiv.lean,Mathlib/Algebra/MvPolynomial/Variables.lean,Mathlib/Analysis/BoxIntegral/Partition/Additive.lean,Mathlib/Analysis/BoxIntegral/Partition/Basic.lean,Mathlib/Analysis/BoxIntegral/Partition/Split.lean,Mathlib/Analysis/Calculus/LagrangeMultipliers.lean,Mathlib/CategoryTheory/Category/PartialFun.lean,Mathlib/Computability/TMToPartrec.lean,Mathlib/Data/Option/Defs.lean,Mathlib/LinearAlgebra/Basis.lean,Mathlib/Logic/Embedding/Set.lean,Mathlib/Logic/Equiv/Basic.lean,Mathlib/MeasureTheory/OuterMeasure/Induced.lean,Mathlib/NumberTheory/Dioph.lean,Mathlib/Topology/Compactness/Paracompact.lean,Mathlib/Topology/LocallyFinite.lean 17 12 ['Ruben-VandeVelde', 'YaelDillies', 'github-actions', 'grunweg', 'urkud'] nobody 1
294-9120
9 months ago
294-84667
9 months ago
7-18420
7 days
11800 JADekker
author:JADekker
feat : Define KappaLindelöf spaces Define KappaLindelöf spaces by following the first one-third of the API for Lindelöf spaces. The remainder will be added in a future PR. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-zulip t-topology merge-conflict please-adopt 301/2 Mathlib.lean,Mathlib/Topology/Compactness/KappaLindelof.lean,Mathlib/Topology/Compactness/Lindelof.lean 3 38 ['ADedecker', 'JADekker', 'PatrickMassot', 'StevenClontz', 'adomani', 'github-actions', 'grunweg', 'kim-em', 'urkud'] nobody 1
266-54938
8 months ago
266-76913
8 months ago
119-10687
119 days
11500 mcdoll
author:mcdoll
refactor(Topology/Algebra/Module/WeakDual): Clean up - Move `Dual` and `dualPairing` lower in the import-hierachy - deduplicate `dualPairing` - Bundle continuity statements to `CLM`s. - Make `WeakDual` and `WeakSpace` reducible - Remove `refine'` in favor of `refine` --- Cleaning up `Analysis/NormedSpace/WeakDual` will be done in a second PR [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology merge-conflict awaiting-author 227/179 Mathlib.lean,Mathlib/Analysis/Fourier/RiemannLebesgueLemma.lean,Mathlib/Analysis/InnerProductSpace/Adjoint.lean,Mathlib/Analysis/InnerProductSpace/Dual.lean,Mathlib/Analysis/LocallyConvex/Polar.lean,Mathlib/Analysis/NormedSpace/Dual.lean,Mathlib/Analysis/NormedSpace/WeakDual.lean,Mathlib/Analysis/VonNeumannAlgebra/Basic.lean,Mathlib/MeasureTheory/Function/AEEqOfIntegral.lean,Mathlib/MeasureTheory/Measure/FiniteMeasure.lean,Mathlib/Topology/Algebra/Module/CharacterSpace.lean,Mathlib/Topology/Algebra/Module/Dual.lean,Mathlib/Topology/Algebra/Module/WeakDual.lean,docs/overview.yaml,docs/undergrad.yaml 15 14 ['ADedecker', 'grunweg', 'j-loreaux', 'kkytola', 'mathlib-bors', 'mcdoll'] nobody 2
244-55902
8 months ago
244-55902
8 months ago
46-5572
46 days
13514 madvorak
author:madvorak
feat(Computability/ContextFreeGrammar): closure under union - [ ] depends on: #15895 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-computability merge-conflict blocked-by-other-PR 448/4 Mathlib/Computability/ContextFreeGrammar.lean 1 50 ['Rida-Hamadani', 'YaelDillies', 'github-actions', 'leanprover-community-mathlib4-bot', 'madvorak'] nobody 1
219-35924
7 months ago
219-35924
7 months ago
72-28392
72 days
12133 ADedecker
author:ADedecker
feat: generalize instIsLowerProd to arbitrary products Also change a bit the proof of the product case to match my own taste, feel free to tell if you prefer the old one. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order t-topology merge-conflict awaiting-author 34/14 Mathlib/Topology/Constructions.lean,Mathlib/Topology/Order/LowerUpperTopology.lean 2 13 ['Ruben-VandeVelde', 'TwoFX', 'github-actions', 'jcommelin', 'mans0954', 'mathlib-bors', 'riccardobrasca'] nobody 2
206-41972
6 months ago
206-41972
6 months ago
63-69206
63 days
17176 arulandu
author:arulandu
feat: integrals and integrability with .re Lemmas for swapping order of .re and integration/integrability. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-measure-probability merge-conflict awaiting-author 49/0 Mathlib/MeasureTheory/Function/L1Space.lean,Mathlib/MeasureTheory/Integral/IntegrableOn.lean,Mathlib/MeasureTheory/Integral/IntervalIntegral.lean,Mathlib/MeasureTheory/Integral/SetIntegral.lean 4 30 ['EtienneC30', 'arulandu', 'github-actions', 'loefflerd'] nobody 1
131-4299
4 months ago
131-4299
4 months ago
9-73631
9 days
2605 eric-wieser
author:eric-wieser
chore: better error message in linarith On this mwe: ```lean import Mathlib.Tactic.Linarith example (s : Set ℕ) (h : s = s) : 0 ≤ 1 := by linarith ``` this now indicates where the internal error is coming from. Is there a better way of chaining errors than this? --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta merge-conflict awaiting-author 12/1 Mathlib/Tactic/Linarith/Preprocessing.lean 1 3 ['Vierkantor', 'harahu', 'kim-em', 'mo271'] nobody 1
130-20459
4 months ago
564-80146
1 year ago
4-7271
4 days
21761 JovanGerb
author:JovanGerb
feat(Algebra): add lemmas `mul_self` and `add_self` This is point (4) in https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Possible.20improvements.20to.20Lean.2FMathlib/near/499085779 I decided to go with `n + n = 2 * n` instead of `n + n = n * 2` because it feels more natural. Feel free to suggest the opposite. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict delegated
label:t-algebra$
206/196 Archive/Imo/Imo1959Q2.lean,Archive/Imo/Imo1961Q3.lean,Archive/Imo/Imo2008Q4.lean,Archive/Imo/Imo2013Q1.lean,Archive/Imo/Imo2024Q3.lean,Archive/MiuLanguage/DecisionSuf.lean,Archive/Wiedijk100Theorems/Partition.lean,Archive/ZagierTwoSquares.lean,Mathlib/Algebra/CharP/Two.lean,Mathlib/Algebra/CharZero/Lemmas.lean,Mathlib/Algebra/Group/Defs.lean,Mathlib/Algebra/Group/Even.lean,Mathlib/Algebra/Lie/Weights/RootSystem.lean,Mathlib/Algebra/Order/Field/Basic.lean,Mathlib/Algebra/Order/Group/Lattice.lean,Mathlib/Algebra/Order/Group/Unbundled/Abs.lean,Mathlib/Algebra/Order/Ring/Basic.lean,Mathlib/Algebra/Order/Ring/Unbundled/Basic.lean,Mathlib/Algebra/Order/Round.lean,Mathlib/Algebra/Polynomial/Taylor.lean,Mathlib/Algebra/Ring/BooleanRing.lean,Mathlib/Algebra/Ring/Defs.lean,Mathlib/Algebra/Ring/Hom/Defs.lean,Mathlib/Algebra/Ring/Int/Parity.lean,Mathlib/Algebra/Ring/Invertible.lean,Mathlib/Algebra/Ring/Parity.lean,Mathlib/Algebra/Ring/SumsOfSquares.lean,Mathlib/Algebra/Symmetrized.lean,Mathlib/Algebra/Tropical/Basic.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Jacobian.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Projective.lean,Mathlib/Analysis/CStarAlgebra/CStarMatrix.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Order.lean,Mathlib/Analysis/Complex/Isometry.lean,Mathlib/Analysis/Complex/PhragmenLindelof.lean,Mathlib/Analysis/Complex/UpperHalfPlane/Metric.lean,Mathlib/Analysis/Convex/Mul.lean,Mathlib/Analysis/Convex/SpecificFunctions/Deriv.lean,Mathlib/Analysis/InnerProductSpace/LinearMap.lean,Mathlib/Analysis/Normed/Lp/ProdLp.lean,Mathlib/Analysis/NormedSpace/MStructure.lean,Mathlib/Analysis/RCLike/Basic.lean,Mathlib/Analysis/SpecialFunctions/Bernstein.lean,Mathlib/Analysis/SpecialFunctions/BinaryEntropy.lean,Mathlib/Analysis/SpecialFunctions/Complex/Arctan.lean,Mathlib/Analysis/SpecialFunctions/Complex/Arg.lean,Mathlib/Analysis/SpecialFunctions/Gamma/Beta.lean,Mathlib/Analysis/SpecialFunctions/Gaussian/GaussianIntegral.lean,Mathlib/Analysis/SpecialFunctions/PolarCoord.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Angle.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Series.lean,Mathlib/Combinatorics/Additive/AP/Three/Defs.lean,Mathlib/Combinatorics/SetFamily/HarrisKleitman.lean,Mathlib/Combinatorics/SimpleGraph/DegreeSum.lean,Mathlib/Combinatorics/SimpleGraph/Matching.lean,Mathlib/Computability/AkraBazzi/AkraBazzi.lean,Mathlib/Computability/Language.lean,Mathlib/Data/Complex/Abs.lean,Mathlib/Data/Complex/Module.lean,Mathlib/Data/Complex/Norm.lean,Mathlib/Data/ENNReal/Holder.lean,Mathlib/Data/ENNReal/Inv.lean,Mathlib/Data/Nat/Bitwise.lean,Mathlib/Data/Nat/Cast/Order/Ring.lean,Mathlib/Data/Nat/Choose/Central.lean,Mathlib/Data/Num/Lemmas.lean,Mathlib/Data/Num/Prime.lean,Mathlib/Data/Real/Pi/Irrational.lean,Mathlib/Data/ZMod/Basic.lean,Mathlib/Dynamics/Circle/RotationNumber/TranslationNumber.lean,Mathlib/FieldTheory/Finite/Basic.lean,Mathlib/Geometry/Euclidean/Angle/Oriented/RightAngle.lean,Mathlib/Geometry/Euclidean/Angle/Unoriented/RightAngle.lean,Mathlib/GroupTheory/Coxeter/Inversion.lean,Mathlib/GroupTheory/Perm/Cycle/Type.lean,Mathlib/GroupTheory/SpecificGroups/Alternating.lean,Mathlib/GroupTheory/SpecificGroups/Dihedral.lean,Mathlib/GroupTheory/SpecificGroups/KleinFour.lean,Mathlib/LinearAlgebra/AffineSpace/Midpoint.lean,Mathlib/LinearAlgebra/Matrix/Charpoly/Eigs.lean,Mathlib/LinearAlgebra/Matrix/PosDef.lean,Mathlib/LinearAlgebra/QuadraticForm/Complex.lean,Mathlib/LinearAlgebra/SesquilinearForm.lean,Mathlib/MeasureTheory/Function/L1Space/HasFiniteIntegral.lean,Mathlib/MeasureTheory/Integral/Bochner.lean,Mathlib/MeasureTheory/Integral/Gamma.lean,Mathlib/MeasureTheory/Measure/LevyProkhorovMetric.lean,Mathlib/NumberTheory/Cyclotomic/Embeddings.lean,Mathlib/NumberTheory/FLT/Three.lean,Mathlib/NumberTheory/GaussSum.lean,Mathlib/NumberTheory/LegendreSymbol/Basic.lean,Mathlib/NumberTheory/LegendreSymbol/JacobiSymbol.lean,Mathlib/NumberTheory/LegendreSymbol/QuadraticChar/Basic.lean,Mathlib/NumberTheory/LegendreSymbol/QuadraticReciprocity.lean,Mathlib/NumberTheory/ModularForms/EisensteinSeries/UniformConvergence.lean,Mathlib/NumberTheory/Multiplicity.lean,Mathlib/NumberTheory/NumberField/Basic.lean,Mathlib/NumberTheory/NumberField/CanonicalEmbedding/ConvexBody.lean,Mathlib/NumberTheory/PellMatiyasevic.lean,Mathlib/NumberTheory/SumPrimeReciprocals.lean 117 13 ['JovanGerb', 'YaelDillies', 'github-actions', 'grunweg', 'mathlib-bors', 'riccardobrasca'] nobody 2
112-82253
3 months ago
113-27024
3 months ago
0-54729
15 hours
17005 YnirPaz
author:YnirPaz
feat(SetTheory/Cardinal/Regular): define singular cardinals Define singular cardinals and prove basic lemmas about them. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-set-theory merge-conflict WIP 94/1 Mathlib.lean,Mathlib/SetTheory/Cardinal/Regular.lean,Mathlib/SetTheory/Ordinal/Basic.lean 3 28 ['YaelDillies', 'YnirPaz', 'github-actions', 'vihdzp'] nobody 1
112-54631
3 months ago
188-47813
6 months ago
34-18388
34 days
18463 vihdzp
author:vihdzp
feat(SetTheory/Ordinal/Notation/FundamentalSequence): define type of fundamental sequences We define `Sequence α` as the type of sequences with length 0, 1, or `ω`, and give a basic API. A subsequent PR will introduce the notion of a (countable and computable) fundamental sequence and establish basic results. The goal of this is to generalize [`ONote.fundamentalSequence`](https://leanprover-community.github.io/mathlib4_docs/Mathlib/SetTheory/Ordinal/Notation.html#ONote.fundamentalSequence) to allow the construction of fundamental sequences for other ordinal notations. --- See [my ordinal notation repository](https://github.com/vihdzp/ordinal-notation/blob/a6fdd7fe7cb521e686ea271902e7e5496f1804d3/OrdinalNotation/Cantor.lean#L1218) for a demonstration of how this API looks in practice. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-set-theory t-order merge-conflict 174/1 Mathlib.lean,Mathlib/SetTheory/Ordinal/Notation/Cantor.lean,Mathlib/SetTheory/Ordinal/Notation/FundamentalSequence.lean 3 19 ['YnirPaz', 'b-mehta', 'github-actions', 'vihdzp'] nobody 1
110-54008
3 months ago
110-54008
3 months ago
52-25108
52 days
15991 vihdzp
author:vihdzp
feat(SetTheory/Ordinal/CantorNormalForm): alternate CNF recursion principle The idea of this recursion principle is that you can build an ordinal by adding one power of `b` at a time, as long as `1 < b ≤ ω`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-set-theory t-logic merge-conflict awaiting-author 43/0 Mathlib/SetTheory/Ordinal/Arithmetic.lean,Mathlib/SetTheory/Ordinal/CantorNormalForm.lean,Mathlib/SetTheory/Ordinal/Exponential.lean 3 8 ['YaelDillies', 'eric-wieser', 'github-actions', 'vihdzp'] nobody 1
83-31960
2 months ago
83-31960
2 months ago
91-50443
91 days
17758 vihdzp
author:vihdzp
feat(SetTheory/Ordinal/ENat): `Ordinal.toENat` We essentially copy the `Cardinal/ENat` file but make it for ordinals instead. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-set-theory merge-conflict 300/0 Mathlib.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/SetTheory/Cardinal/ENat.lean,Mathlib/SetTheory/Ordinal/Arithmetic.lean,Mathlib/SetTheory/Ordinal/Basic.lean,Mathlib/SetTheory/Ordinal/ENat.lean 6 2 ['Command-Master', 'github-actions', 'vihdzp'] nobody 1
83-31489
2 months ago
83-31489
2 months ago
126-40106
126 days
15915 vihdzp
author:vihdzp
chore(SetTheory/Ordinal/CantorNormalForm): `CNF.exponents` and `CNF.coeffs` We rewrite theorems about the Cantor Normal Form in terms of their lists of exponents and coefficients, instead of awkwardly talking about their first and second entries. We also put all theorems about the CNF in its own namespace. This keeps us from cluttering the `Ordinal` namespace, and it also avoids having to prefix everything by `CNF_` constantly. --- - [x] depends on: #16998 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-set-theory t-logic merge-conflict awaiting-author 117/44 Mathlib/SetTheory/Ordinal/CantorNormalForm.lean 1 32 ['Command-Master', 'YaelDillies', 'YnirPaz', 'digama0', 'github-actions', 'mathlib4-dependent-issues-bot', 'vihdzp'] nobody 1
80-62087
2 months ago
80-62087
2 months ago
53-79724
53 days
19189 YnirPaz
author:YnirPaz
feat(SetTheory/Ordinal/Arithmetic): order isomorphism between omega and the natural numbers --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-set-theory merge-conflict awaiting-author 44/0 Mathlib/Order/SuccPred/Limit.lean,Mathlib/SetTheory/Ordinal/Arithmetic.lean 2 21 ['YaelDillies', 'YnirPaz', 'github-actions', 'vihdzp'] nobody 1
80-61842
2 months ago
80-61842
2 months ago
47-37012
47 days
19275 eric-wieser
author:eric-wieser
fix: if nolint files change, do a full rebuild Otherwise CI will succeed when removing entries from the file, but fail later when someone changes something unrelated. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict delegated 8/0 lakefile.lean 1 20 ['YaelDillies', 'adomani', 'eric-wieser', 'github-actions', 'grunweg', 'mathlib-bors'] nobody 1
66-20303
2 months ago
66-20303
2 months ago
0-214
3 minutes
23411 PatrickMassot
author:PatrickMassot
chore: remove finiteness from Order.Filter.Lift Co-authored-by: Anatole Dedecker --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) longest-pole t-topology merge-conflict 48/21 Mathlib/Dynamics/TopologicalEntropy/DynamicalEntourage.lean,Mathlib/Order/Filter/Basic.lean,Mathlib/Order/Filter/Finite.lean,Mathlib/Order/Filter/Lift.lean,Mathlib/Order/Filter/SmallSets.lean,Mathlib/Topology/Algebra/ContinuousMonoidHom.lean,Mathlib/Topology/Basic.lean 7 4 ['Vierkantor', 'github-actions', 'kim-em', 'leanprover-community-bot-assistant'] nobody 1
62-38370
2 months ago
62-57939
2 months ago
10-21608
10 days
19425 hrmacbeth
author:hrmacbeth
perf: gcongr forward-reasoning adjustment This PR changes the "forward-reasoning" component of `gcongr`, rendering it more efficient, particularly in problems with a large number of variables/hypotheses in the context. Previously `gcongr` attempted to match *every* `LocalDecl` against *every* node in the parse tree using *each* of the five implemented `@[gcongr_forward]` mini-tactics: matching directly, matching after applying `symm`, matching after applying `le_of_lt`, etc etc. The new algorithm filters out the non-Prop `LocalDecl`s, and also adjusts the `@[gcongr_forward]` extensions so that, rather than re-apply the relevant lemmas (`symm`, `le_of_lt`, etc) at every node in the parse tree, the lemmas are applied in advance to the `LocalDecl`s and the result (if successful) stored. The performance effect on mathlib as a whole is miniscule, but it speeds up the profiler's count of "tactic execution of Mathlib.Tactic.GCongr" in the newly-added test from 257 ms to 47 ms, and has a similar effect on real-life examples in an analysis project of mine. Co-authored-by: Mario Carneiro --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) (Note that Mario provided the ideas but not the code, so please review with appropriate diligence!) merge-conflict awaiting-author 130/59 Mathlib/Order/Lattice.lean,Mathlib/Tactic/GCongr/Core.lean,Mathlib/Tactic/GCongr/ForwardAttr.lean,MathlibTest/GCongr/inequalities.lean 4 17 ['Vierkantor', 'github-actions', 'hrmacbeth', 'leanprover-bot', 'leanprover-community-bot-assistant'] Vierkantor
assignee:Vierkantor
1
60-36821
1 month ago
60-36823
1 month ago
4-16654
4 days
12673 grunweg
author:grunweg
feat: add ContDiff.lipschitzOnWith A C¹ function is Lipschitz on each convex compact set. From sphere-eversion. -------- Commits can be reviewed independently. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis merge-conflict awaiting-author help-wanted 30/11 Mathlib/Analysis/Calculus/ContDiff/RCLike.lean 1 6 ['Ruben-VandeVelde', 'github-actions', 'grunweg', 'sgouezel'] nobody 1
53-16899
1 month ago
53-16899
1 month ago
1-7552
1 day
18893 vihdzp
author:vihdzp
feat(Order/InitialSeg): `InitialSeg.exists_relIso_sum` If `r` is an initial segment of `s`, there exists some other relation `t` with `Sum.Lex r t ≃r s`. --- - [x] depends on: #17989 - [ ] depends on: #20409 The names `sumLexLtLE` and `sumLexLeLT` are very sketch, and better suggestions are welcome. Likewise it'd be cool if anyone can figure out how to golf these results. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order merge-conflict awaiting-author blocked-by-other-PR 102/10 Mathlib/Order/InitialSeg.lean,Mathlib/Order/RelIso/Basic.lean,Mathlib/Order/RelIso/Set.lean,Mathlib/SetTheory/Ordinal/Basic.lean 4 13 ['YaelDillies', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'vihdzp'] nobody 1
47-25576
1 month ago
47-25578
1 month ago
46-65043
46 days
8370 eric-wieser
author:eric-wieser
refactor(Analysis/NormedSpace/Exponential): remove the `𝕂` argument from `exp` This argument is still needed for almost all the lemmas, which means it can longer be found by unification. We keep around `expSeries 𝕂 A`, as it's needed for talking about the radius of convergence over different base fields. This is a prerequisite for #8372, as we can't merge the functions until they have the same interface.\ Zulip thread: [#mathlib4 > Real.exp @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Real.2Eexp/near/401602245) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) This is started from the mathport output on https://github.com/leanprover-community/mathlib/pull/19244 awaiting-zulip t-analysis merge-conflict 432/387 Mathlib/Analysis/CStarAlgebra/Exponential.lean,Mathlib/Analysis/CStarAlgebra/Spectrum.lean,Mathlib/Analysis/Normed/Algebra/Exponential.lean,Mathlib/Analysis/Normed/Algebra/MatrixExponential.lean,Mathlib/Analysis/Normed/Algebra/QuaternionExponential.lean,Mathlib/Analysis/Normed/Algebra/Spectrum.lean,Mathlib/Analysis/Normed/Algebra/TrivSqZeroExt.lean,Mathlib/Analysis/NormedSpace/DualNumber.lean,Mathlib/Analysis/SpecialFunctions/ContinuousFunctionalCalculus/ExpLog.lean,Mathlib/Analysis/SpecialFunctions/Exponential.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Series.lean 11 29 ['YaelDillies', 'eric-wieser', 'girving', 'github-actions', 'j-loreaux', 'kbuzzard', 'leanprover-community-bot-assistant', 'urkud'] nobody 1
45-69965
1 month ago
57-12195
1 month ago
29-60989
29 days
19315 quangvdao
author:quangvdao
feat(Data/Finsupp/Fin): Add `Finsupp` operations on `Fin` tuple This PR adds more analogues of operations on `Fin` tuples to the `Finsupp` setting. Before, there were only `Finsupp.cons` and `Finsupp.tail`. Now there are also `Finsupp.snoc`, `Finsupp.insertNth`, `Finsupp.init`, and `Finsupp.removeNth`. These all come with supporting lemmas. I also removed the porting comment about `succAboveCases` in `Data/Fin/Basic`, and added a lemma about `succAbove` in `Data/Fin/Tuple/Basic`. --- - [x] depends on: #20361 - [x] depends on: #20771 - [x] depends on: #20770 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data merge-conflict awaiting-author 193/16 Mathlib/Algebra/BigOperators/Fin.lean,Mathlib/Algebra/BigOperators/Finsupp.lean,Mathlib/Algebra/MvPolynomial/Equiv.lean,Mathlib/Data/Finsupp/Fin.lean,Mathlib/RingTheory/MvPolynomial/Homogeneous.lean,scripts/nolints_prime_decls.txt 6 44 ['YaelDillies', 'github-actions', 'j-loreaux', 'kbuzzard', 'mathlib4-dependent-issues-bot', 'quangvdao'] nobody 1
33-79826
1 month ago
33-79826
1 month ago
43-81255
43 days
21751 vihdzp
author:vihdzp
refactor(SetTheory/Ordinal/Arithmetic): rework `Ordinal.pred` API This PR does the following: - give a simpler definition of `Ordinal.pred` - replace `¬ ∃ a, o = succ a` and `∀ a, o ≠ succ a` by `IsSuccPrelimit o` throughout - improve theorem names --- There's a legitimate question of whether we even want `Ordinal.pred` (see [Zulip](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Ordinal.2Epred)) but this should be a good change in the meanwhile regardless. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-set-theory maintainer-merge merge-conflict 102/67 Mathlib/SetTheory/Ordinal/Arithmetic.lean,Mathlib/SetTheory/Ordinal/Exponential.lean 2 13 ['YaelDillies', 'github-actions', 'grunweg', 'vihdzp'] nobody 1
33-79798
1 month ago
80-58425
2 months ago
36-50134
36 days
7907 urkud
author:urkud
feat: introduce `NthRoot` notation class Also use it for `Real.sqrt`, and replace the few occurrences of `sqrt` that do not already use the notation. --- [Zulip](https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/.60Sqrt.60.20notation.20typeclass/near/400086502) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-analysis awaiting-CI merge-conflict
label:t-algebra$
193/156 Archive/Imo/Imo1959Q2.lean,Archive/Imo/Imo1960Q2.lean,Archive/Imo/Imo2001Q2.lean,Archive/Imo/Imo2006Q3.lean,Archive/Imo/Imo2008Q3.lean,Archive/Imo/Imo2008Q4.lean,Archive/Sensitivity.lean,Archive/Wiedijk100Theorems/AreaOfACircle.lean,Mathlib.lean,Mathlib/Algebra/NthRoot.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Instances.lean,Mathlib/Analysis/Complex/AbelLimit.lean,Mathlib/Analysis/RCLike/Basic.lean,Mathlib/Analysis/SpecialFunctions/Pow/Asymptotics.lean,Mathlib/Analysis/SpecialFunctions/Pow/Real.lean,Mathlib/Analysis/SpecialFunctions/Stirling.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Basic.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Bounds.lean,Mathlib/Data/Real/GoldenRatio.lean,Mathlib/Data/Real/Sqrt.lean,Mathlib/LinearAlgebra/Matrix/PosDef.lean,Mathlib/MeasureTheory/Measure/Lebesgue/VolumeOfBalls.lean,Mathlib/NumberTheory/Harmonic/GammaDeriv.lean,Mathlib/NumberTheory/NumberField/CanonicalEmbedding/ConvexBody.lean,Mathlib/NumberTheory/NumberField/ClassNumber.lean,Mathlib/NumberTheory/NumberField/Discriminant/Basic.lean,Mathlib/Probability/Distributions/Gaussian.lean,MathlibTest/positivity.lean 28 9 ['eric-wieser', 'github-actions', 'kmill', 'urkud'] nobody 1
32-20540
1 month ago
286-34098
9 months ago
0-0
0 seconds
17027 vihdzp
author:vihdzp
feat(SetTheory/ZFC/Ordinal): von Neumann hierarchy of sets --- - [x] depends on: #16996 - [x] depends on: #17016 - [x] depends on: #17026 - [x] depends on: #18239 - [ ] depends on: #19946 - [x] depends on: #19967 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-set-theory merge-conflict 204/29 Mathlib.lean,Mathlib/SetTheory/Ordinal/Basic.lean,Mathlib/SetTheory/ZFC/Basic.lean,Mathlib/SetTheory/ZFC/Neumann.lean,Mathlib/SetTheory/ZFC/Rank.lean 5 8 ['alreadydone', 'github-actions', 'mathlib4-dependent-issues-bot', 'vihdzp'] nobody 1
31-13200
1 month ago
31-13202
1 month ago
0-344
5 minutes
13685 niklasmohrin
author:niklasmohrin
feat(Combinatorics): add definitions for network flows Although we might not have any super-interesting results ready for mathlib yet, I feel that the definitions from this commit are already mature enough to include. These definitions are ported from last semester's work we did at https://github.com/niklasmohrin/lean-seminar-2023 and I have put some time in to refactor our code to `Int` and now to any parameter `R`. In the linked repository, there is some more stuff that I can send in. One obstacle without integer values is that it is not clear why a maximum flow would exist. I think the best way to tackle this would be to prove max-flow-min-cut theorem and implement the Ford-Fulkerson algorithm. It has been pointed out on Zulip that there is an [Isabelle formalization of the Edmonds Karp Algorithm](https://www.isa-afp.org/entries/EdmondsKarp_Maxflow.html). I feel that the definitions are pretty solid and it makes sense to include them, even if just for unifying definitions across downstream projects. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-combinatorics merge-conflict awaiting-author 244/0 Mathlib.lean,Mathlib/Combinatorics/Flow/Basic.lean,docs/references.bib 3 57 ['Shreyas4991', 'YaelDillies', 'b-mehta', 'github-actions', 'leanprover-community-bot-assistant', 'madvorak', 'niklasmohrin'] nobody 1
25-70063
25 days ago
25-70065
25 days ago
86-21072
86 days
17129 joneugster
author:joneugster
feat(Tactic/Linter): add unicode linter for unicode variant-selectors Unicode characters can be followed by one of the two "variant-selectors" `\FE0E` (text) or `\FE0F` (emoji). These appear to the user as a single unicode character and they might copy them by accident. For example `✅️` (`\u2705\uFE0F`), `✅` (`\u2705`) and `✅︎` (`\u2705\uFE0E`) are three variants of the "same" unicode character. The one without variant-selector might display as either emoji or not, depending on the user's device and font. Add unicode linter ensuring variant-selector only appear on specified characters and also ensuring these characters always have the correct variant selector to avoid confusions. Everything flagged by this linter can be fixed fully automatically with `lake exe lint-style --fix` or by commenting `bot fix style` on the PR. --- - tracking PR: #16215 ## Zulip discussions: - https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/Whitelist.20for.20Unicode.3F - https://leanprover.zulipchat.com/#narrow/stream/113488-general/topic/Lean.20specific.20font ## Related PRs: - leanprover/lean4#5015 added some emoji-variant selectors to Emojis used in `Lean` itself. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-linter merge-conflict delegated awaiting-author 245/14 Mathlib.lean,Mathlib/GroupTheory/GroupExtension/Defs.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter/TextBased.lean,Mathlib/Tactic/Linter/UnicodeLinter.lean,Mathlib/Tactic/Widget/Calc.lean,Mathlib/Tactic/Widget/CongrM.lean,Mathlib/Tactic/Widget/Conv.lean,Mathlib/Tactic/Widget/GCongr.lean,Mathlib/Topology/ContinuousMap/Weierstrass.lean,MathlibTest/LintStyleTextBased.lean 11 25 ['YaelDillies', 'adomani', 'github-actions', 'grunweg', 'joneugster', 'kim-em', 'leanprover-community-bot-assistant'] nobody 1
24-14325
24 days ago
24-14327
24 days ago
82-54712
82 days
21476 grunweg
author:grunweg
feat(lint-style): enable running on downstream projects Enable lint-style to run on downstream projects, by making the following modifications: - allow passing an explicit list of libraries to lint: if nothing is passed, it lints `Mathlib`, `Archive` and `Counterexamples` (as before); otherwise, it lints precisely the passed modules - only check init imports, undocumented scripts and the errors from `lint-style.py` when linting Mathlib - make the style exceptions file configurable and optional: using the `nolints-file` flag, the exceptions file can be configured. If the flag is omitted, we try to find a file at `scripts/nolints-style.txt` --- and otherwise proceed with no style exceptions. This means mathlib can continue unchanged, and downstream projects can either add an explicit exceptions file, or proceed without any exceptions. After this PR, one should be able to run lint-style on a downstream project by `lake exe lint-style ProjectName`. Prompted by [this zulip discussion](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/lint-style.20for.20downstream.20libraries). --- - [ ] depends on: #24570 - [ ] depends on: #24953 (I did not test the last part.) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-linter merge-conflict 58/19 Mathlib/Tactic/Linter/TextBased.lean,scripts/lint-style.lean 2 19 ['Vierkantor', 'adomani', 'github-actions', 'grunweg', 'joneugster', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] joneugster
assignee:joneugster
1
14-27655
14 days ago
14-27658
14 days ago
43-17409
43 days
24965 erdOne
author:erdOne
refactor: Make `IsLocalHom` take unbundled map --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) maintainer-merge t-algebra merge-conflict awaiting-author
label:t-algebra$
16/7 Mathlib/Algebra/Group/Units/Hom.lean,Mathlib/AlgebraicGeometry/Scheme.lean,Mathlib/Geometry/RingedSpace/LocallyRingedSpace.lean,Mathlib/Geometry/RingedSpace/LocallyRingedSpace/HasColimits.lean,Mathlib/Geometry/RingedSpace/OpenImmersion.lean 5 6 ['alreadydone', 'erdOne', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant'] nobody 1
6-62766
6 days ago
6-62767
6 days ago
10-26015
10 days
24789 Ruben-VandeVelde
author:Ruben-VandeVelde
chore: move Algebra.Group.Hom.End to Algebra.Ring --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-algebra merge-conflict awaiting-author
label:t-algebra$
55/50 Mathlib.lean,Mathlib/Algebra/Group/Hom/End.lean,Mathlib/Algebra/Group/Hom/Instances.lean,Mathlib/Algebra/Module/End.lean,Mathlib/Algebra/Ring/Hom/End.lean 5 6 ['Ruben-VandeVelde', 'YaelDillies', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant'] nobody 1
0-5911
1 hour ago
0-5913
1 hour ago
0-1530
25 minutes

All open PRs

Number Author Title Description Labels +/- Modified files (first 100) 📝 💬 All users who commented or reviewed Assignee(s) Updated Last status change total time in review
8978 eric-wieser
author:eric-wieser
perf: add `extends flat` to all hom classes I expect that [lean4#2905](https://github.com/leanprover/lean4/pull/2905) will cause this to have worse performance. --- - [ ] depends on: #8977 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR WIP 119/36 Mathlib/Algebra/Algebra/Equiv.lean,Mathlib/Algebra/Algebra/Hom.lean,Mathlib/Algebra/Algebra/NonUnitalHom.lean,Mathlib/Algebra/Group/Hom/Defs.lean,Mathlib/Algebra/Order/Hom/Monoid.lean,Mathlib/Algebra/Order/Hom/Ring.lean,Mathlib/Algebra/Ring/CentroidHom.lean,Mathlib/Algebra/Ring/Hom/Defs.lean,Mathlib/Algebra/Star/StarAlgHom.lean,Mathlib/Data/FunLike/Basic.lean,Mathlib/GroupTheory/GroupAction/Hom.lean,Mathlib/Order/Heyting/Hom.lean,Mathlib/Order/Hom/Bounded.lean,Mathlib/Order/Hom/CompleteLattice.lean,Mathlib/Order/Hom/Lattice.lean,Mathlib/RingTheory/Jacobson.lean,Mathlib/Topology/Algebra/ContinuousMonoidHom.lean,Mathlib/Topology/Order/Hom/Basic.lean,Mathlib/Topology/Order/Hom/Esakia.lean 19 5 ['eric-wieser', 'leanprover-bot', 'leanprover-community-mathlib4-bot'] nobody
377-45937
1 year ago
377-45989
1 year ago
0-0
0 seconds
14727 jjaassoonn
author:jjaassoonn
feat(RingTheory/Flat/CategoryTheory): a flat module has vanishing higher Tor groups [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra awaiting-author
label:t-algebra$
37/1 Mathlib/RingTheory/Flat/CategoryTheory.lean 1 3 ['github-actions', 'kim-em'] nobody
313-42773
10 months ago
326-79221
10 months ago
3-28223
3 days
14583 lecopivo
author:lecopivo
fix: make concrete cycle notation local fix: make c[...] notation for concrete cycles local --- The notation for concrete cycles prevents you using `c[i]` notation for `c : Array _` This currently does not work ``` import Mathlib variable (c : Array Nat) (i : Fin c.size) #check c[i] -- breaks because of notation for concrete cycles ``` This PR just marks it as local to prevent this issue. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author 1/1 Mathlib/GroupTheory/Perm/Cycle/Concrete.lean 1 2 ['eric-wieser', 'github-actions'] nobody
313-42773
10 months ago
334-78023
10 months ago
0-12793
3 hours
14345 digama0
author:digama0
feat: the Dialectica category is monoidal closed - [x] depends on: #14274 The monoidal closed structure of the Dialectica category. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory awaiting-author 252/0 Mathlib.lean,Mathlib/CategoryTheory/Dialectica/Closed.lean 2 3 ['github-actions', 'kim-em', 'leanprover-community-mathlib4-bot'] nobody
313-42772
10 months ago
329-10776
10 months ago
12-17890
12 days
14386 Parcly-Taxel
author:Parcly-Taxel
feat: the Rado graph --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics WIP 163/0 Mathlib.lean,Mathlib/Combinatorics/SimpleGraph/Rado.lean 2 1 ['github-actions'] nobody
313-42772
10 months ago
341-23940
11 months ago
0-0
0 seconds
14444 digama0
author:digama0
fix(GeneralizeProofs): unreachable! bug As [reported on Zulip](https://leanprover.zulipchat.com/#narrow/stream/270676-lean4/topic/Unreachable.20code.20reached.20in.20Lean.204.2E8.2E0/near/449286780). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta awaiting-author 1/1 Mathlib/Tactic/GeneralizeProofs.lean 1 4 ['github-actions', 'jcommelin', 'kmill'] nobody
313-42772
10 months ago
328-80342
10 months ago
10-36842
10 days
12952 adomani
author:adomani
test: length statistics --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) test-ci WIP 124/0 .github/workflows/mathlib_stats.yml,.github/workflows/ml_stats_label.yaml,scripts/mathlib_stats.sh 3 9 ['github-actions'] nobody
313-42771
10 months ago
342-15451
11 months ago
0-0
0 seconds
13036 joelriou
author:joelriou
feat(CategoryTheory/Sites): under certain conditions, cover preserving functors preserve 1-hypercovers Previously, in order to show that a functor between Grothendieck sites was continuous, it was necessary to show that it was "cover preserving" and "compatible preserving". There were two lemmas which could be used in order to show that a functor was "compatible preserving". Since #13012, the better condition of "1-hypercover preserving" functor was introduced and it implies that the functor is continuous. In this PR, under the same assumptions as in the two lemmas mentionned above, we show that cover preserving functors are 1-hypercover preserving functors. This gives slightly better criteria in order to show that a functor is continuous. --- - [x] depends on: #13004 - [x] depends on: #13011 - [x] depends on: #13012 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory WIP 94/7 Mathlib/CategoryTheory/Sites/Continuous.lean,Mathlib/CategoryTheory/Sites/CoverPreserving.lean,Mathlib/CategoryTheory/Sites/Over.lean,Mathlib/CategoryTheory/Sites/Sieves.lean 4 2 ['github-actions', 'leanprover-community-mathlib4-bot'] nobody
313-42770
10 months ago
339-85492
11 months ago
0-0
0 seconds
12452 JADekker
author:JADekker
feat(Cocardinal) : add some more api Just a small PR to add a bit more API for cocardinal filters. Not everything seems to generalise nicely from cofinite, so I didn't include such results. Currently the file has one `sorry`, I'm not sure how to complete this proof. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology awaiting-CI 75/0 Mathlib/Order/Filter/Cocardinal.lean 1 0 [] nobody
313-42770
10 months ago
335-23470
11 months ago
0-0
0 seconds
12984 adomani
author:adomani
Adomani/periodic reports dev custom action --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) test-ci WIP 366/0 .github/workflows/mathlib_stats.yml,.github/workflows/ml_stats_label.yaml,scripts/count_decls.lean,scripts/mathlib_stats.sh 4 n/a ['github-actions'] nobody
313-42770
10 months ago
unknown
unknown
11991 adomani
author:adomani
draft: syntax data linter A linter that prints `SyntaxNodeKind`s and `Range`s for all the nodes of a command. See this [Zulip discussion](https://leanprover.zulipchat.com/#narrow/stream/217875-Is-there-code-for-X.3F/topic/undocumented.20things). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP 152/0 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/SyntaxDataLinter.lean 3 0 [] nobody
313-42769
10 months ago
342-15444
11 months ago
0-0
0 seconds
12006 adomani
author:adomani
feat: the `suffa` tactic The `suffa` tactic. `suffa tac` runs the tactic sequence `tac` and returns a `Try this:` suggestion of the form `suffices [target_after_tac] by tac; assumption`. For example ```lean example {m n : Nat} (h : m = n) : 0 + m = n := by suffa rewrite [Nat.zero_add] assumption ``` suggests the replacement ```lean example {m n : Nat} (h : m = n) : 0 + m = n := by suffices m = n by rewrite [Nat.zero_add] assumption assumption ``` See [this thread](https://leanprover.zulipchat.com/#narrow/stream/113488-general/topic/Try.20this.3A.20suffices.20simpa) as well as [this message](https://leanprover.zulipchat.com/#narrow/stream/144837-PR-reviews/topic/.2311822.20flexible.20tactics.20linter/near/431895664). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta awaiting-author 161/0 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Suffa.lean,test/Suffa.lean 4 1 ['YaelDillies'] nobody
313-42769
10 months ago
368-30727
1 year ago
58-85902
58 days
10998 hmonroe
author:hmonroe
feat(Logic): Arithmetization of partial recursive functions (toward Gödel's first incompleteness theorem) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-logic awaiting-author 364/0 Mathlib.lean,Mathlib/Logic/Godel/PartArith.lean 2 3 ['Ruben-VandeVelde', 'YaelDillies'] nobody
313-42768
10 months ago
368-14004
1 year ago
97-20483
97 days
10099 mcdoll
author:mcdoll
feat: Integration by parts for higher dimensional spaces --- - [x] depends on: #9987 - [x] depends on: #10105 - [x] depends on: #10107 - [x] depends on: #10115 - [x] depends on: #10118 - [x] depends on: #10182 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-measure-probability t-analysis WIP 429/0 Mathlib/Analysis/InnerProductSpace/OrthoDecomp.lean,Mathlib/MeasureTheory/Integral/test2.lean 2 3 ['alexjbest', 'github-actions', 'leanprover-community-mathlib4-bot'] nobody
313-42768
10 months ago
486-73185
1 year ago
0-0
0 seconds
9469 dupuisf
author:dupuisf
feat: maximum modulus principle for functions vanishing at infinity This PR adds versions of the maximum modulus principle for functions vanishing at infinity that parallel those we already had for functions over a bounded set. These will have applications in e.g. norm interpolation. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis awaiting-author 71/0 Mathlib/Analysis/Complex/AbsMax.lean 1 8 ['dupuisf', 'j-loreaux'] nobody
313-42767
10 months ago
507-84013
1 year ago
12-86009
12 days
9320 BoltonBailey
author:BoltonBailey
chore: Golf simp calls This script runs on a lean file or directory of lean files, and removes unnecessary lemmas from simp calls in those files. Some comments I have received about how this should work: - [ ] It should not do anything if it changes the InfoView environment, since people may have added unnecessary lemmas that make the InfoView easier to read. - [ ] It should not make any changes that make compilation slower, since some lemmas may be present for perf reasons. - [ ] It should be written in Lean rather than Python. I should look into dwrensha's [`TryAtEachStep`](https://github.com/dwrensha/tryAtEachStep) for an example of a project that analyzes tactic-by-tactic changes to a file. TODOs: - [ ] Specific golfs: - [ ] Per @alreadydone: simp only [] could be replaced by dsimp only - [ ] Remove lemmas in calls to `simp` as well as `simp only`. - [ ] Replace `simp only` with `simp_rw`. - [ ] Replace `simp_rw` with `rw` where possible. - [ ] Replace `rw [...] ; rw [...]` with one call to `rw`, and same for `simp` and friends. - [ ] More advanced: - [ ] Just delete tokens/lines/tactics willy-nilly and see if that finds anything. - [ ] Fine-tune an LLM on reviewer suggestions from Mathlib PRs. Successor to #9079. This PR focuses on removing lemmas from simp calls. It only does this for terminal simp/simp only, to avoid changing intermediate states. #9101 looks to add more features. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP 151/0 scripts/golf.py 1 1 ['BoltonBailey'] nobody
313-42767
10 months ago
401-75134
1 year ago
0-0
0 seconds
9510 eric-wieser
author:eric-wieser
feat(Analysis/Calculus/DualNumber): Extending differentiable functions to dual numbers This shows that this operation preserves multiplication and composition --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-analysis awaiting-CI WIP
label:t-algebra$
119/0 Mathlib/Analysis/Calculus/DualNumber.lean 1 4 ['github-actions'] nobody
313-42767
10 months ago
519-30798
1 year ago
0-0
0 seconds
9352 chenyili0818
author:chenyili0818
feat: arithmetic lemmas for `gradient` This file is based on Mathlib.Analysis.Calculus.Gradient.Basic, and describes the calculation properties Co-authored-by: Ziyu Wang [tropicalfish910@gmail.com](mailto:tropicalfish910@gmail.com) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis awaiting-author 404/0 Mathlib.lean,Mathlib/Analysis/Calculus/Gradient/Lemmas.lean 2 30 ['chenyili0818', 'github-actions', 'jcommelin', 'sgouezel', 'winstonyin'] nobody
313-42767
10 months ago
475-23932
1 year ago
51-80670
51 days
8224 Kha
author:Kha
chore: add `lean4checker` benchmark WIP 16/0 scripts/bench/temci-config.run.yml 1 3 ['Kha', 'grunweg', 'kim-em', 'leanprover-bot'] nobody
313-42766
10 months ago
381-9295
1 year ago
0-0
0 seconds
7890 grhkm21
author:grhkm21
feat(Mathlib/Tactic/Setm): implement setm tactic This is my first time doing metaprogramming in Lean 4, please provide feedback when you have them :) The `setm` tactic, which stands for `set` + matching, matches a given expression with the goal and introduces new local hypotheses for the named holes specified. One of the best usage is for rearrangement proofs. As a simple example, ```lean example : (1 + 1) + (4 * 3) - (1 + 1) = (3 * 4 : Rat) := by setm ?A + ?B - ?A = (?C : Rat) rw [show ∀ A B, A + B - A = B by intro A B ; ring_nf ] apply Rat.mul_comm ``` One can imagine replacing the three term expression with a 7 term algebraic expression. This was developed with tons of help from [Zulip](https://leanprover.zulipchat.com/#narrow/stream/239415-metaprogramming-.2F-tactics/topic/Help.20with.20writing.20tactic), especially from Thomas. Thanks! TODO: - [X] Support `setm ... at ...` syntax, see *example 1* below - [X] Write docs - [ ] Use `withNewMCtxDepth` - [X] Rename the intermediate `MVar`s, see *example 2* below - [ ] Use `elabTermWithHolesPostponing` in conjunction with `Term.synthesizeSyntheticMVarsNoPostPoning` after `isDefEq` to handle instances Example 1: ```lean /- Usage with `using` and `at` keywords -/ example (h1 : 1 + 1 = 3) (h2 : 1 + 3 = 5) (h3 : 2 + 2 = 5) : true := by setm ?A + _ = (?B : Nat) using h2 at h1 h2 h3 guard_hyp A := 1 guard_hyp B := 5 guard_hyp h1 : A + A = 3 guard_hyp h2 : A + 3 = B guard_hyp h3 : 2 + 2 = B trivial ``` Example 2: ```lean /- Test reusing named holes -/ example (h : b + a = c) : a + b = c := by /- setm 1-/ setm ?A + ?B = (_ : Nat) guard_hyp A := a guard_hyp B := b /- clean up -/ unfold_let A B clear hA hB A B /- setm 2 -/ rewrite [Nat.add_comm] setm ?A + ?B = (_ : Nat) at h ⊢ guard_hyp A := b guard_hyp B := a exact h ``` Co-authored-by: Jireh Loreaux [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta 141/0 Mathlib.lean,Mathlib/Tactic/Common.lean,Mathlib/Tactic/Setm.lean,test/Setm.lean 4 3 ['thorimur'] nobody
313-42766
10 months ago
594-44290
1 year ago
0-0
0 seconds
7125 eric-wieser
author:eric-wieser
feat: additive monoid structure via biproducts I suspect I'm missing a trick with these transport lemmas. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory awaiting-CI WIP 237/0 Mathlib/CategoryTheory/Limits/Skeleton.lean 1 2 ['alreadydone', 'eric-wieser'] nobody
313-42766
10 months ago
623-30507
1 year ago
0-0
0 seconds
6859 MohanadAhmed
author:MohanadAhmed
TryLean4Bundle: Windows Bundle Creator # `TryLean4Bundle`: Windows Bundle Creator A Windows batch script and a CI yml file that create an self extracting archive. The user should 1. just download the archive, 2. double click the archive to expand 3. double click the `RunLean.bat` script in the expanded archive. The script currently downloads 7 dependencies into CI then unpacks them in the appropriate locations and finally packs them back. To try a bundle created using these scripts but from a different repo see (https://github.com/MohanadAhmed/TryLean4Bundle/releases) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) CI WIP help-wanted 114/0 .github/workflows/mk_windows_bundle.yml,scripts/windowsBundle.bat 2 0 [] nobody
313-42766
10 months ago
649-72037
1 year ago
0-0
0 seconds
4786 thorimur
author:thorimur
feat: AppBuilder utils This supplements `Lean.Meta.AppBuilder`, introducing variants of `mkAppN` and `mkAppM` which allow for more fine-grained management of existing and created metavariables. [Description pending] --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta 205/0 Mathlib.lean,Mathlib/Lean/Meta/AppBuilder.lean 2 0 [] nobody
313-42765
10 months ago
733-43119
2 years ago
0-0
0 seconds
5745 alexjbest
author:alexjbest
feat: a tactic to consume type annotations, and make constructor nicer During the copenhagen masterclass I found some situations where applying the constructor tactic left the goal in a difficult to read state when autoParams were present. We add a simple tactic to clean these up, and a macro for `constructor` to behave more like the constructor notation and do this automatically (constructor is in core) It seems that these things should be cleaned up by simp, but a simp lemma to remove these annotations is not accepted by lean as the types are too similar. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta awaiting-author 41/0 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Consume.lean,test/consume.lean 4 4 ['alexjbest', 'digama0', 'kim-em', 'kmill'] nobody
313-42765
10 months ago
398-6259
1 year ago
51-33797
51 days
15224 AnthonyBordg
author:AnthonyBordg
feat(CategoryTheory/Sites): covering families and their associated Grothendieck topology Define covering families on a category and their associated Grothendieck topology by using the API for `Coverage`. Give an explicit characterization of the covering sieves of the said topology. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-category-theory awaiting-author 112/0 Mathlib.lean,Mathlib/CategoryTheory/Sites/CoveringFamilies.lean 2 20 ['AnthonyBordg', 'adamtopaz', 'dagurtomas', 'github-actions', 'joelriou'] nobody
308-17782
10 months ago
313-11447
10 months ago
1-48443
1 day
15453 tomaz1502
author:tomaz1502
Track formalization of runtime complexity I finished porting https://github.com/leanprover-community/mathlib3/pull/14494/ to Lean 4 and made several small PRs, as suggested. This meta PR is used to track the progress of the smaller PRs. ## Pending PRs - [Formalization of List.insertionSort](https://github.com/leanprover-community/mathlib4/pull/15449) - [Lemmas about Split](https://github.com/leanprover-community/mathlib4/pull/15450) - [Formalization of List.merge](https://github.com/leanprover-community/mathlib4/pull/15451) - [Formalization of List.mergeSort](https://github.com/leanprover-community/mathlib4/pull/15452) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 525/0 Mathlib.lean,Mathlib/Computability/Timed/InsertionSort.lean,Mathlib/Computability/Timed/Merge.lean,Mathlib/Computability/Timed/MergeSort.lean,Mathlib/Computability/Timed/Split.lean 5 4 ['joneugster', 'mergify'] nobody
299-37050
9 months ago
299-37104
9 months ago
0-0
0 seconds
14009 grunweg
author:grunweg
chore: replace continuity -> fun_prop in remaining directories After the current set of PRs, the only continuity remnants either need more attention or are merely for tagging continuity lemmas. --- - [x] depends on: #11092 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis awaiting-author 6/4 Mathlib/Computability/AkraBazzi/AkraBazzi.lean,Mathlib/LinearAlgebra/AffineSpace/ContinuousAffineEquiv.lean 2 4 ['github-actions', 'j-loreaux', 'leanprover-community-mathlib4-bot'] nobody
298-43126
9 months ago
298-43126
9 months ago
6-67481
6 days
14563 awueth
author:awueth
feat: if-then-else of exclusive or statement --- If `¬(P ∧ Q)` then `ite (P ∨ Q) a 1 = (ite P a 1) * (ite Q a 1)` [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra awaiting-author
label:t-algebra$
5/0 Mathlib/Algebra/Group/Basic.lean 1 3 ['eric-wieser', 'github-actions', 'kim-em'] nobody
298-35158
9 months ago
298-35158
9 months ago
6-38745
6 days
14733 jjaassoonn
author:jjaassoonn
feat(RingTheory/Flat/CategoryTheory): a module is flat iff tensoring preserves finite limits --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra awaiting-author
label:t-algebra$
99/1 Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Basic.lean,Mathlib/Algebra/Category/ModuleCat/Monoidal/RightExact.lean,Mathlib/RingTheory/Flat/CategoryTheory.lean 4 2 ['github-actions', 'kim-em'] nobody
298-33109
9 months ago
298-33109
9 months ago
6-6256
6 days
12103 BoltonBailey
author:BoltonBailey
feat: Berlekamp-Welch Implementation of the Berlekamp-Welch Decoding procedure, and proof of its correctness within the decoding radius. Todos: - [ ] Integrate with coding theory part of library - [ ] Gaussian Elimination lives in `Mathlib/Tactic/Linarith/SimplexAlgorithm/Gauss.lean`, may need facts about it. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra WIP
label:t-algebra$
78/0 Mathlib/Algebra/Polynomial/BerlekampWelch.lean 1 0 [] nobody
298-32654
9 months ago
298-32654
9 months ago
0-0
0 seconds
9406 wupr
author:wupr
feat: Inverse limits of modules, abelian groups, and rings --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra WIP
label:t-algebra$
174/0 Mathlib/Algebra/InverseLimit.lean 1 8 ['alreadydone', 'erdOne', 'wupr'] nobody
298-32507
9 months ago
298-32507
9 months ago
0-0
0 seconds
11106 BoltonBailey
author:BoltonBailey
feat: file for lemmas about MvPolynomials over NoZeroDivisors WIP See discussion from #11073 --- - [x] depends on: #11095 - [x] depends on: #11094 - [ ] depends on: #12664 [We need this lemma to establish fact about degreeOf n (p + q)] [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra blocked-by-other-PR WIP
label:t-algebra$
85/0 Mathlib/Algebra/MvPolynomial/NoZeroDivisors.lean 1 1 ['leanprover-community-mathlib4-bot'] nobody
298-32351
9 months ago
298-32351
9 months ago
0-0
0 seconds
9040 BoltonBailey
author:BoltonBailey
feat: `to_snoc` an attribute for generating lemmas with snoc in them This is an experimental PR for a new attribute which is basically `to_additive`, but instead of changing multiplication to addition, it changes `cons` to `snoc`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta please-adopt WIP help-wanted 1292/0 Mathlib/Tactic/ToSnoc.lean 1 0 [] nobody
298-32307
9 months ago
298-32307
9 months ago
0-0
0 seconds
10387 adomani
author:adomani
feat(Tactic/ComputeDegree): add `polynomial` tactic Introducing the `polynomial` tactic, summing up `compute_degree, monicity` and adding support for `leadingCoeff`. This is more of a proof of concept: if there is interest in this tactic, I can polish it up. See [this Zulip discussion](https://leanprover.zulipchat.com/#narrow/stream/113489-new-members/topic/Compute.20roots.20of.20polynomials/near/420713624). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) RFC t-meta WIP 24/0 Mathlib/Tactic/ComputeDegree.lean 1 0 [] nobody
298-32306
9 months ago
298-32306
9 months ago
0-0
0 seconds
9693 madvorak
author:madvorak
feat: Linear programming in the standard form --- Zulip discussion: https://leanprover.zulipchat.com/#narrow/stream/144837-PR-reviews/topic/.237386.20Linear.20Programming Four PRs incompatible with each other: https://github.com/leanprover-community/mathlib4/pull/7386 (list of constraints) https://github.com/leanprover-community/mathlib4/pull/9693 (matrix form) https://github.com/leanprover-community/mathlib4/pull/10026 (Antoine Chambert-Loir's def; semirings, linear) https://github.com/leanprover-community/mathlib4/pull/10159 (Antoine Chambert-Loir's def; rings, affine) - [x] depends on: #9652 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra RFC WIP
label:t-algebra$
86/0 Mathlib.lean,Mathlib/LinearAlgebra/Matrix/LinearProgramming.lean 2 14 ['apurvanakade', 'github-actions', 'leanprover-community-mathlib4-bot', 'madvorak'] nobody
298-32221
9 months ago
298-32221
9 months ago
0-0
0 seconds
7386 madvorak
author:madvorak
feat: Define linear programs Linear programs over a general `Module` with constraints given in the form "aᵀx - b ≥ 0" and the objective function as an `AffineMap` to be minimized. --- Zulip discussion: https://leanprover.zulipchat.com/#narrow/stream/144837-PR-reviews/topic/.237386.20Linear.20Programming Four PRs incompatible with each other: https://github.com/leanprover-community/mathlib4/pull/7386 (list of constraints) https://github.com/leanprover-community/mathlib4/pull/9693 (matrix form) https://github.com/leanprover-community/mathlib4/pull/10026 (Antoine Chambert-Loir's def; semirings, linear) https://github.com/leanprover-community/mathlib4/pull/10159 (Antoine Chambert-Loir's def; rings, affine) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra RFC WIP
label:t-algebra$
87/0 Mathlib.lean,Mathlib/LinearAlgebra/LinearProgramming.lean 2 63 ['Shreyas4991', 'YaelDillies', 'eric-wieser', 'github-actions', 'kim-em', 'madvorak'] nobody
298-31831
9 months ago
298-31831
9 months ago
66-6720
66 days
7322 BoltonBailey
author:BoltonBailey
feat: Default list Generalizes `ListBlank` to use a specified default, rather than the one supplied by `Inhabited`, with an eye to using this type to represent computable polynomials. This is a forward port of this [mathlib 3 PR](https://github.com/leanprover-community/mathlib/pull/16160) TODOs: - [ ] Replace ListBlank in TuringMachine.lean with this (see comment below) - [ ] Make sure imports are minimal and alphabetical --- - [x] depends on: #7307 - [x] depends on: #7323 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-computability please-adopt WIP 600/0 Mathlib/Computability/ListBlank.lean 1 3 ['BoltonBailey', 'leanprover-community-mathlib4-bot', 'urkud'] nobody
298-31811
9 months ago
298-31811
9 months ago
0-0
0 seconds
7219 Ruben-VandeVelde
author:Ruben-VandeVelde
feat: Equivs for AddMonoidAlgebras --- Extracted from #6718. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra awaiting-author
label:t-algebra$
113/0 Mathlib.lean,Mathlib/Algebra/MonoidAlgebra/Equiv.lean 2 12 ['Ruben-VandeVelde', 'alreadydone', 'eric-wieser'] eric-wieser
assignee:eric-wieser
298-31793
9 months ago
298-31794
9 months ago
0-0
0 seconds
13163 erdOne
author:erdOne
feat(.vscode/module-docstring.code-snippet): Prevent auto-complete from firing on `do` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta awaiting-author 5/0 .vscode/module-docstring.code-snippets 1 5 ['erdOne', 'grunweg', 'robertylewis', 'trivial1711'] nobody
298-30620
9 months ago
298-30620
9 months ago
50-50444
50 days
10026 madvorak
author:madvorak
Linear programming according to Antoine Chambert-Loir's book --- Zulip discussion: https://leanprover.zulipchat.com/#narrow/stream/144837-PR-reviews/topic/.237386.20Linear.20Programming Four PRs incompatible with each other: https://github.com/leanprover-community/mathlib4/pull/7386 (list of constraints) https://github.com/leanprover-community/mathlib4/pull/9693 (matrix form) https://github.com/leanprover-community/mathlib4/pull/10026 (Antoine Chambert-Loir's def; semirings, linear) https://github.com/leanprover-community/mathlib4/pull/10159 (Antoine Chambert-Loir's def; rings, affine) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra RFC WIP
label:t-algebra$
86/0 Mathlib.lean,Mathlib/LinearAlgebra/LinearProgramming.lean 2 9 ['eric-wieser', 'madvorak', 'riccardobrasca'] nobody
297-9684
9 months ago
297-9684
9 months ago
0-0
0 seconds
10159 madvorak
author:madvorak
Linear programming according to Antoine Chambert-Loir's book — affine version --- Zulip discussion: https://leanprover.zulipchat.com/#narrow/stream/144837-PR-reviews/topic/.237386.20Linear.20Programming Four PRs incompatible with each other: https://github.com/leanprover-community/mathlib4/pull/7386 (list of constraints) https://github.com/leanprover-community/mathlib4/pull/9693 (matrix form) https://github.com/leanprover-community/mathlib4/pull/10026 (Antoine Chambert-Loir's def; semirings, linear) https://github.com/leanprover-community/mathlib4/pull/10159 (Antoine Chambert-Loir's def; rings, affine) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra RFC WIP
label:t-algebra$
83/0 Mathlib.lean,Mathlib/LinearAlgebra/LinearProgramming.lean 2 7 ['eric-wieser', 'madvorak', 'riccardobrasca'] nobody
297-9670
9 months ago
297-9670
9 months ago
0-0
0 seconds
11890 adomani
author:adomani
feat: the terminal refine linter A linter that warns on usages of `refine` and `refine'` as a finishing tactic. See this [Zulip discussion](https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/Usage.20of.20refine'). ### Conclusion of the experiment Systematic replacements of terminal `refine` with `exact` leads to an overall slow-down. --- - [ ] depends on: #15616 (disable the linter in downstream projects) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-linter awaiting-author 77/0 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter/TerminalRefineLinter.lean 3 14 ['adomani', 'github-actions', 'grunweg', 'joneugster', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'urkud'] nobody
294-43251
9 months ago
294-43253
9 months ago
18-13508
18 days
11207 luigi-massacci
author:luigi-massacci
feat(Topology/MetricSpace): Add new file with type of Katetov maps add a type of Katetov maps (one point extensions of a metric) and related notation and FunLike coercions. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-topology WIP 138/0 Mathlib.lean,Mathlib/Topology/MetricSpace/Katetov.lean,docs/references.bib 3 16 ['fpvandoorn', 'jcommelin', 'kim-em', 'luigi-massacci', 'urkud'] nobody
294-19535
9 months ago
396-21620
1 year ago
26-83567
26 days
11090 pangelinos
author:pangelinos
feat: define spectral spaces and prove that a quasi-compact open of a spectral space is spectral Define spectral spaces and prove that a quasi-compact open of a spectral space is spectral. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-topology please-adopt good first issue 69/0 Topology/Spectral/basic.lean 1 15 ['YaelDillies', 'adomani', 'j-loreaux', 'jcommelin', 'kim-em', 'pangelinos'] nobody
294-19410
9 months ago
298-32336
9 months ago
16-44803
16 days
9795 sinhp
author:sinhp
feat: the type `Fib` of fibre of a function at a point This is the most basic file of the theory of fibred categories developed here: https://github.com/sinhp/LeanFibredCategories/tree/master --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory awaiting-author 74/0 Mathlib.lean,Mathlib/Data/Fiber.lean 2 17 ['adri326', 'joelriou', 'sinhp'] nobody
292-22186
9 months ago
507-41653
1 year ago
1-32924
1 day
15055 sinhp
author:sinhp
feat: the category of pointed objects of a concrete category This file defines the category of pointed objects of a concrete category. After this we will have the categories of pointed groups, pointed abelian groups, pointed groupoids, etc. To define `Pointed.functor`, we need to add the following "pullback" construction to the category of elements. ``` @[simps obj map] def pullback (F : D ⥤ Type w) (G : C ⥤ D) : (G ⋙ F).Elements ⥤ F.Elements where obj X := ⟨G.obj X.1, X.2⟩ map {X Y} f := ⟨G.map f.1, f.2⟩ ``` This is called pullback since the display map of `G ⋙ F` (i.e. `π (G ⋙ F)`) is a pullback of the display map of `F`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory awaiting-author 185/0 Mathlib.lean,Mathlib/CategoryTheory/ConcreteCategory/Pointed.lean,Mathlib/CategoryTheory/Elements.lean 3 13 ['dagurtomas', 'github-actions', 'kim-em'] nobody
291-29903
9 months ago
313-30559
10 months ago
7-80557
7 days
15786 Multramate
author:Multramate
feat(AlgebraicGeometry/EllipticCurve/NumberField/Height): define heights on Weierstrass curves --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebraic-geometry t-number-theory WIP 650/0 Mathlib/AlgebraicGeometry/EllipticCurve/NumberField/Height.lean 1 2 ['Multramate', 'github-actions'] nobody
290-38431
9 months ago
299-77361
9 months ago
0-0
0 seconds
11385 BoltonBailey
author:BoltonBailey
feat: scripts to analyze overlap between namespaces TODOs: - [ ] Translate to Lean - [ ] Put in Utils directory --- - [x] depends on: #12322 [When this is rewritten in Lean, it would be good to output data in the form of a table] [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta WIP 86/0 scripts/RecordNamespaces.lean,scripts/namespace-overlap.py 2 1 ['leanprover-community-mathlib4-bot'] nobody
284-20715
9 months ago
unknown
unknown
16253 Shreyas4991
author:Shreyas4991
feat: Basics of Discrete Fair Division in Mathlib This PR adds the basics of discrete fair division in mathlib. We include the definitions of allocations, valuations, properties of valuations, and the following notions : Envy-Freeness (EF), Envy-Freeness upto 1 good (EF1), and envy freeness upto any good (EFX). We also include the various implications between these notions. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author WIP 144/0 Mathlib/GameTheory/FairDivision/Discrete/Basic.lean 1 9 ['Shreyas4991', 'eric-wieser', 'github-actions'] nobody
284-1952
9 months ago
284-1952
9 months ago
0-20853
5 hours
14669 Command-Master
author:Command-Master
feat(Data/Nat/PartENat): add lemmas for PartENat Add some missing lemmas for `PartENat`, as well as the additive homomorphism from it to `WithTop Int`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data new-contributor awaiting-author 90/0 Mathlib/Data/Nat/PartENat.lean 1 3 ['erdOne', 'github-actions', 'urkud'] nobody
281-31957
9 months ago
281-31957
9 months ago
0-0
0 seconds
15121 Eloitor
author:Eloitor
feat: iff theorems for IsSplitEpi and IsSplitMono in opposite category --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-category-theory awaiting-author 40/0 Mathlib/CategoryTheory/EpiMono.lean 1 3 ['github-actions', 'joelriou', 'mattrobball'] nobody
280-81302
9 months ago
312-40561
10 months ago
7-3203
7 days
15895 madvorak
author:madvorak
feat(Computability/ContextFreeGrammar): mapping between two types of nonterminal symbols --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-computability WIP 172/0 Mathlib/Computability/ContextFreeGrammar.lean 1 43 ['YaelDillies', 'github-actions', 'madvorak'] nobody
280-11695
9 months ago
284-45204
9 months ago
1-43047
1 day
12278 Rida-Hamadani
author:Rida-Hamadani
feat(Combinatorics/SimpleGraph): Provide iff statements for distance equal and greater than 2 I need these lemmas to prove that Moore graphs of girth 5 are strongly regular. --- - [x] depends on: #11945 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics awaiting-author 76/0 Mathlib/Combinatorics/SimpleGraph/Metric.lean 1 2 ['github-actions', 'leanprover-community-mathlib4-bot'] nobody
279-66821
9 months ago
279-66821
9 months ago
1-68738
1 day
16570 yuma-mizuno
author:yuma-mizuno
chore(Tactic/CategoryTheory): change `TermElabM` to `MetaM` Separated from #15335. To use `Qq`, we need to modify `Qq` to support universe matching. See [Zulip](https://leanprover.zulipchat.com/#narrow/stream/144837-PR-reviews/topic/.2315335.20meta.20code.20for.20monoidal.20categories). --- - [ ] depends on: #15335 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta WIP 26/15 Mathlib/Tactic/CategoryTheory/BicategoryCoherence.lean,Mathlib/Tactic/CategoryTheory/Coherence.lean 2 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mergify'] nobody
273-18561
9 months ago
273-63809
9 months ago
0-0
0 seconds
10591 adri326
author:adri326
feat(Topology/Algebra/ConstMulAction): properties of continuous actions in Hausdorff spaces Defines some useful properties of `ContinuousConstSMul` group actions on Hausdorff spaces: - `MulAction.isClosed_fixedBy`, which proves that the `fixedBy α m` set is closed - `t2_separation_smul`, which constructs an open set `s` such that `s` and `g • s` are disjoint - `Set.InjOn.t2_separation_smul`, the extension of `t2_separation_smul` to a set of group elements whose action is injective --- This PR belongs my series of PR around the formalization of Rubin's theorem. `MulAction.isClosed_fixedBy` is used in several places along the proof, and the separation lemmas are primarily used in showing that `(fixedBy α g)ᶜ` and `(fixedBy α h)ᶜ` are disjoint under some intricate but fully group-theoretic condition. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-topology awaiting-author
label:t-algebra$
57/0 Mathlib/Topology/Algebra/ConstMulAction.lean 1 9 ['ADedecker', 'adri326', 'j-loreaux', 'jcommelin'] ADedecker
assignee:ADedecker
272-10553
8 months ago
424-23291
1 year ago
55-82183
55 days
14704 Command-Master
author:Command-Master
feat(FieldTheory): define typeclass for simple extensions, and prove some properties Define `SimpleExtension F K`, which says that `K` is a simple field extension of `F`, and show that together with transcendentality it implies `IsFractionRing F[X] K`. --- - [x] depends on: #14710 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra awaiting-author WIP
label:t-algebra$
120/0 Mathlib.lean,Mathlib/FieldTheory/SimpleExtension.lean 2 17 ['Command-Master', 'acmepjz', 'github-actions', 'leanprover-community-mathlib4-bot', 'tb65536'] nobody
267-38003
8 months ago
267-38003
8 months ago
0-0
0 seconds
16773 arulandu
author:arulandu
feat(Probability/Distributions): formalize Beta distribution Formalize Beta distribution, using Gamma distribution as a reference. Added real-valued beta wrapper, in the manner of gamma. Thanks to @EtienneC30 for help with casting real <-> complex. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-measure-probability awaiting-author 286/1 Mathlib.lean,Mathlib/Analysis/SpecialFunctions/Gamma/Beta.lean,Mathlib/Probability/Distributions/Beta.lean 3 48 ['EtienneC30', 'arulandu', 'github-actions', 'vihdzp'] arulandu
assignee:arulandu
262-41519
8 months ago
267-38237
8 months ago
1-21124
1 day
14237 js2357
author:js2357
feat: Define the localization of a fractional ideal at a prime ideal Define the localization of a fractional ideal at a prime ideal, and prove some basic properties. --- This PR is part 3 out of 4 of a proof of `isDedekindDomain_iff_isDedekindDomainDvr`. Part 4 is available here: #14242 - [x] depends on: #14099 Part 1 - [x] depends on: #14216 Part 2 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra awaiting-author
label:t-algebra$
230/0 Mathlib.lean,Mathlib/RingTheory/FractionalIdeal/LocalizedAtPrime.lean,Mathlib/RingTheory/Localization/Basic.lean 3 20 ['Vierkantor', 'YaelDillies', 'github-actions', 'js2357', 'kbuzzard', 'leanprover-community-mathlib4-bot'] Vierkantor
assignee:Vierkantor
258-20363
8 months ago
258-20481
8 months ago
26-39463
26 days
16041 vihdzp
author:vihdzp
feat(SetTheory/Ordinal/Arithmetic): `Ordinal.toNat` A simple function sending ordinals less than `ω` to themselves, and anything else to `0`. --- - [ ] depends on: #17758 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-set-theory t-logic awaiting-author blocked-by-other-PR WIP 58/0 Mathlib/SetTheory/Ordinal/Arithmetic.lean 1 4 ['github-actions', 'mathlib4-dependent-issues-bot', 'urkud', 'vihdzp'] nobody
237-55814
7 months ago
237-55816
7 months ago
54-31491
54 days
10796 mcdoll
author:mcdoll
feat(Tactic/Positivity): non-negativity of functions --- This makes the `Finset.sum` and `integral_nonneg` extensions even more useful. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta WIP 27/0 Mathlib/Tactic/Positivity/Core.lean 1 1 ['YaelDillies'] nobody
232-41934
7 months ago
474-34003
1 year ago
0-0
0 seconds
14603 awueth
author:awueth
feat: degree is invariant under graph isomorphism --- Mathlib has the definition `SimpleGraph.Iso.mapNeighborSet` which is an equivalence between neighbor sets induced by an isomorphism. Would it be beneficial to add the same equivalence for `neighborFinset`? [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-combinatorics WIP 24/0 Mathlib/Combinatorics/SimpleGraph/Map/Finite.lean 1 11 ['awueth', 'github-actions', 'jcommelin', 'kim-em', 'urkud'] nobody
230-13904
7 months ago
230-13904
7 months ago
31-44440
31 days
18630 tomaz1502
author:tomaz1502
feat(Computability.Timed): Formalization of runtime complexity of List.mergeSort This PR adds the formalization of the runtime complexity of the merge sort algorithm, defined in `Data/List/Sort`. Requires: https://github.com/leanprover-community/mathlib4/pull/15451 References: - Previous PR on mathlib3: https://github.com/leanprover-community/mathlib3/pull/14494/ - First discussion on Zulip: https://leanprover.zulipchat.com/#narrow/stream/113488-general/topic/BSc.20Final.20Project/near/220647062 - Second disussion on Zulip: https://leanprover.zulipchat.com/#narrow/stream/113488-general/topic/Formalization.20of.20Runtime.20Complexity.20of.20Sorting.20Algorithms/near/284184450 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-computability new-contributor 526/0 Mathlib.lean,Mathlib/Computability/Timed/InsertionSort.lean,Mathlib/Computability/Timed/Merge.lean,Mathlib/Computability/Timed/MergeSort.lean,Mathlib/Computability/Timed/Split.lean 5 8 ['github-actions'] nobody
216-10463
7 months ago
216-10463
7 months ago
0-0
0 seconds
18472 FR-vdash-bot
author:FR-vdash-bot
perf: lower the priority of `Comm*.to*` instances `CommRing.toRing` is an exception. `CommRing` is so important that it needs to be looked up early. An important goal of #7873 is also to search for `Zero/One/Add/Mul` instances first along `Zero/One/Add/Mul` -> ... -> `Ring` -> `CommRing` -> `Field`. --- - [ ] depends on: #18474 - [ ] depends on: #18641 From #7873. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-bench slow-typeclass-synthesis t-algebra blocked-by-other-PR
label:t-algebra$
33/10 Mathlib/Algebra/Group/Defs.lean,Mathlib/Algebra/GroupWithZero/Defs.lean,Mathlib/Algebra/Ring/Defs.lean,Mathlib/AlgebraicGeometry/Cover/Open.lean,Mathlib/Data/Int/Cast/Defs.lean,Mathlib/Data/Nat/Cast/Defs.lean,Mathlib/LinearAlgebra/Matrix/Charpoly/Coeff.lean,Mathlib/NumberTheory/LegendreSymbol/GaussEisensteinLemmas.lean,Mathlib/NumberTheory/NumberField/Discriminant/Defs.lean,Mathlib/NumberTheory/Padics/PadicNumbers.lean,Mathlib/NumberTheory/Zsqrtd/QuadraticReciprocity.lean,Mathlib/RingTheory/Filtration.lean,Mathlib/RingTheory/Localization/Integral.lean,Mathlib/Topology/MetricSpace/Polish.lean 14 5 ['FR-vdash-bot', 'github-actions', 'leanprover-bot', 'mathlib4-dependent-issues-bot'] nobody
214-78489
7 months ago
215-3668
7 months ago
0-258
4 minutes
18464 FR-vdash-bot
author:FR-vdash-bot
perf: lower the priority of `toMul` and `toAdd` instances A subsequent PR will try to swap the priorities of `Semigroup.toMul` and `MulOneClass.toMul` to see if it gets better. --- - [ ] depends on: #18472 From #7873. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-bench slow-typeclass-synthesis t-algebra blocked-by-other-PR
label:t-algebra$
38/12 Mathlib/Algebra/BigOperators/Ring/List.lean,Mathlib/Algebra/Group/Defs.lean,Mathlib/Algebra/GroupWithZero/Defs.lean,Mathlib/Algebra/Ring/Defs.lean,Mathlib/Algebra/Ring/Ext.lean 5 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
214-62502
7 months ago
221-74724
7 months ago
0-8515
2 hours
16801 awainverse
author:awainverse
feat(ModelTheory/Equivalence): The quotient type of formulas modulo a theory Defines `FirstOrder.Language.Theory.Formula`: `T.Formula α` is the quotient of `L.Formula α` by equivalence modulo a theory `T`. Puts a boolean algebra instance on `T.Formula α`, with `≤` corresponding to implication. --- - [x] depends on: #16799 - [x] depends on: #16800 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-logic awaiting-author 174/60 Mathlib/ModelTheory/Complexity.lean,Mathlib/ModelTheory/Equivalence.lean,Mathlib/ModelTheory/Types.lean 3 29 ['YaelDillies', 'awainverse', 'github-actions', 'mathlib4-dependent-issues-bot', 'metinersin'] YaelDillies
assignee:YaelDillies
211-80120
6 months ago
220-33539
7 months ago
29-26213
29 days
15809 archiebrowne
author:archiebrowne
feat(RingTheory/MvPolynomial/Ideal): introduce new lemmas about MvPolynomial Ideals Four new lemmas about MvPolynomialIdeals `sub_span_span_sub`, `span_eq_iff_basis_sub`, `mem_basis_mem_span`, `mem_span_exists_dvd_mem_basis`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra awaiting-author
label:t-algebra$
38/0 Mathlib/RingTheory/MvPolynomial/Ideal.lean 1 6 ['Ruben-VandeVelde', 'github-actions', 'riccardobrasca'] riccardobrasca
assignee:riccardobrasca
203-16688
6 months ago
258-18608
8 months ago
41-7533
41 days
6042 MohanadAhmed
author:MohanadAhmed
feat(LinearAlgebra/Matrix/SVD): Singular Value Decomposition of R or C Matrices This file provides proves the SVD theorem which decomposes a real/complex matrix into left eigenvectors, singular values block diagonal matrix and right eigenvectors. Any matrix A (M × N) with rank r = A.rank and with elements in ℝ or ℂ fields can be decompsed into the product of three matrices: $$A = USV$$ * The three matrices are defined as - $U$: an M × M matrix containing the left eigenvectors of the matrix - $S$: an M × N matrix with an r × r block in the upper left corner with nonzero singular values - $V$: an N × N matrix containing the right eigenvectors of the matrix Note that * $S$ is a block matrix $S = [S₁₁, S₁₂; S₂₁, S₂₂]$ with - $S₁₁$: a diagonal r × r matrix and - $S₁₂$ : r × (N - r) zero matrix, S₂₁ : (M - r) × r zero matrix and - $S₂₂$: (M - r) × (N - r) zero matrix * $U$ is a block column matrix U = [U₁ U₂] with - $U₁$ : a M × r containing left eigenvectors with nonzero singular values. - $U₂$ : a M × (M - r) containing left eigenvectors with zero singular values. * $V$ is a block column matrix V = [V₁ V₂] with - $V₁$ : a N × r containing right eigenvectors with nonzero singular values. - $V₂$ : a M × (M - r) containing right eigenvectors with zero singular values. Since in mathlib the eigenvalues of hermitian matrices are defined in an "arbitrary" undetermined order, we begin by partition the singular values into zero and non-zero values. We partition the corresponding eigenvectors from AᴴA and AAᴴ using similar rearrangements. These are included in `SVD.svdReindex`. The basic API for Column and Row partitioned matrices is from `ColumnRowPartitioned`. We then proceed to transfer some of the lemmas we need about eigenvector matrices (for example that they are unitary: i.e. inverse is conjugate transpose.). Note that since invertibility in mathlib is defined for square matrices while our matrices are partitioned i.e. N × (N₁ ⊕ N₂) and N ≃ (N ⊕ N₂), Lean cannot apply the Invertible definition. We workaround this were necessary. Lemma `reduced_spectral_theorem` (`reduced_spectral_theorem'`) shows that AᴴA and AAᴴ, can be reduced to products containing only the non-zero singular eigenvectors. This is later used in proving the main SVD theroem. A few lemmas are provided about the invertibility of the non-zero singular values matrix: `svdσ_inv`, `σ_inv_μ_σ_inv_eq_one`, `IsUnit_det_svdσ`, `IsUnit_det_svdσ_mapK` and `svdσ_inv_mapK`. To make relating left eigenvectors to right eigenvectors easier we define U₁ = AV₁σ⁻¹ while U₂ is obtained from the eigenvectors of (AAᴴ). This avoid a lengthy reindexing operation with many proofs. The vectors in U₂ have no such issue since they are multiplied by zero singular values anyway. Co-authored-by: Mohanad Ahmed --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra please-adopt WIP
label:t-algebra$
588/0 Mathlib.lean,Mathlib/LinearAlgebra/Matrix/SVD/Defs.lean,Mathlib/LinearAlgebra/Matrix/SVD/Reindex.lean 3 114 ['MohanadAhmed', 'Vierkantor', 'alexjbest', 'eric-wieser', 'j-loreaux', 'jcommelin', 'sgouezel'] nobody
203-6254
6 months ago
203-6264
6 months ago
181-72917
181 days
11820 eric-wieser
author:eric-wieser
feat(Algebra/Star/Unitary): add unitarySubgroup --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra awaiting-author
label:t-algebra$
44/0 Mathlib/Algebra/Star/Unitary.lean 1 5 ['eric-wieser', 'j-loreaux'] j-loreaux
assignee:j-loreaux
203-5072
6 months ago
428-54619
1 year ago
5-19391
5 days
19329 adomani
author:adomani
perf(CI): automatically benchmark PRs when they are opened This action posts the comment ``` !bench This is an automated bench-marking that runs when a PR is opened. No need to repeat. ``` whenever a PR is *opened*. It then ignores any subsequent changes to the PR. The automatic benching should help in catching PRs that unknowingly introduce a high performance cost, as was the case for my PR #18033. ### Note. Running `!bench` strains the benchmarking system and it is not feasible to run it on every push. However, Sebastian, in private communication with Johan, approved of automatically benching every PR once, when it is opened. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) CI WIP 25/0 .github/workflows/first_bench_is_free.yml 1 12 ['Ruben-VandeVelde', 'adomani', 'alreadydone', 'eric-wieser', 'github-actions', 'grunweg', 'jcommelin'] nobody
198-45957
6 months ago
200-34912
6 months ago
0-1356
22 minutes
18876 GabinKolly
author:GabinKolly
feat(ModelTheory/Fraisse): add proof that Fraïssé limits exist Fraïssé limits exist. --- All the preparatory work done in other files is contained in the pull request #18749, this pull request adds the work done in ModelTheory/Fraisse, the definition of the sequence of structures whose limit will be the Fraïssé limit, lemmas about this sequence, and then the proof that the limit is indeed a Fraïssé limit. - [ ] depends on: #18749 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-logic blocked-by-other-PR 666/5 Mathlib/ModelTheory/Bundled.lean,Mathlib/ModelTheory/DirectLimit.lean,Mathlib/ModelTheory/FinitelyGenerated.lean,Mathlib/ModelTheory/Fraisse.lean,Mathlib/ModelTheory/PartialEquiv.lean,Mathlib/ModelTheory/Substructures.lean 6 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
184-26420
6 months ago
210-16390
6 months ago
0-37
37 seconds
19972 jjdishere
author:jjdishere
feat(RingTheory): Perfectoid Field We define perfectoid field and its tilt. Mimicking Polish space, we define `PerfectoidField` and `ValuedPerfectoidField`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-analysis t-topology WIP
label:t-algebra$
150/0 Mathlib/RingTheory/Perfectoid.lean 1 1 ['github-actions'] nobody
176-56869
5 months ago
176-56946
5 months ago
0-0
0 seconds
20029 FrederickPu
author:FrederickPu
Allow for Config attributes to be set directly Allow for Config attributes to be set directly when using initialize_simp_projection as per issue #19895 Basically modified initialize_simp_projection so that the user has the option of specifying a tuple of config option values. Ex: ``` initialize_simp_projection MulEquiv (toFun → apply, invFun → symm_apply) (fullyApplied := false) ``` These config options are then converted into projections.  --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-meta WIP 34/4 Mathlib/Tactic/Simps/Basic.lean 1 10 ['FrederickPu', 'YaelDillies', 'fpvandoorn', 'github-actions'] nobody
172-85146
5 months ago
173-33855
5 months ago
0-34081
9 hours
19721 urkud
author:urkud
feat (WIP): formalize Moreira's version of Sard's theorem --- I'm in the process of migrating development to https://github.com/urkud/SardMoreira [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis 427/1 Mathlib.lean,Mathlib/Analysis/Calculus/ContDiff/Defs.lean,Mathlib/Analysis/Calculus/ContDiff/FTaylorSeries.lean,Mathlib/Analysis/Calculus/ContDiff/FaaDiBruno.lean,Mathlib/Analysis/Calculus/Moreira2001.lean 5 1 ['github-actions'] nobody
171-71037
5 months ago
176-67852
5 months ago
0-0
0 seconds
18236 joelriou
author:joelriou
feat(Algebra/Category/ModuleCat/Presheaf): the endofunctor of presheaves of modules induced by an oplax natural transformation An endomorphism of ` ModuleCat.restrictScalarsPseudofunctor`, i.e. a "compatible" family of functors `ModuleCat A ⥤ ModuleCat A` for all (commutative) rings `A` induces a functor `PresheafOfModules R ⥤ PresheafOfModules R` for any presheaf of (commutative) rings `R`. In #18262, this is applied to the construction of exterior powers of a presheaves of modules. --- - [x] depends on: #18197 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-category-theory WIP
label:t-algebra$
180/0 Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Presheaf/FunctorOfNatTrans.lean 2 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
171-7088
5 months ago
171-7126
5 months ago
0-0
0 seconds
20208 js2357
author:js2357
feat: Define the localization of a fractional ideal at a prime ideal Define the localization of a fractional ideal at a prime ideal, and prove some basic properties. --- Alternate version of #14237 generalized to use `IsLocalization` and `IsFractionRing` rather than `Localization.AtPrime` and `FractionRing` [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra WIP
label:t-algebra$
248/0 Mathlib.lean,Mathlib/RingTheory/FractionalIdeal/LocalizedAtPrime.lean 2 1 ['github-actions'] nobody
167-79542
5 months ago
167-79542
5 months ago
0-21
21 seconds
20428 madvorak
author:madvorak
feat(Data/Sign): lemmas about `∈ Set.range SignType.cast` --- Perhaps `in_set_range_singType_cast_iff_abs` needs to be moved somewhere downstream. t-data WIP 40/0 Mathlib/Data/Sign.lean 1 9 ['eric-wieser', 'github-actions', 'madvorak'] nobody
157-2749
5 months ago
157-35152
5 months ago
0-0
0 seconds
20459 Ruben-VandeVelde
author:Ruben-VandeVelde
chore: fix names of roots_C_mul_X_{add,sub}_C_of_IsUnit --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra awaiting-author
label:t-algebra$
11/5 Mathlib/Algebra/Polynomial/FieldDivision.lean,Mathlib/Algebra/Polynomial/Roots.lean 2 2 ['eric-wieser', 'github-actions'] nobody
152-11990
5 months ago
152-11990
5 months ago
4-64422
4 days
10977 grunweg
author:grunweg
feat: germs of smooth functions Define the space of germs of smooth functions (between manifolds). Endow it with a ring structure if the target manifold is a smooth ring (e.g., a Lie group or a field). From the sphere eversion project, rewritten by me. Co-authored-by: Patrick Massot ------- Particular questions for review - is the authorship/copyright information appropriate? (`PatrickMassot` created the file `SmoothGerm` which I adapted; I didn't trace this far back through sphere-eversion.) - is providing all the intermediate algebraic structures (such as, an additive subgroup) on the space of smooth germs useful in practice? (The sphere eversion project only needs a ring structure.) - any further particular API lemmas (e.g., around coercions) which would be good to add? --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis t-topology t-differential-geometry awaiting-author 150/0 Mathlib.lean,Mathlib/Geometry/Manifold/Algebra/SmoothGerm.lean 2 33 ['YaelDillies', 'github-actions', 'grunweg', 'jcommelin', 'kim-em', 'mcdoll'] fpvandoorn
assignee:fpvandoorn
151-86147
5 months ago
286-21112
9 months ago
144-63944
144 days
13483 adomani
author:adomani
feat: automatically replace deprecations This PR introduces `lake exe update_deprecations` that uses the cache to automatically replace deprecated declarations with the corresponding un-deprecated one. The script handles namespacing, replacing a possibly non-fully-qualified, deprecated name with the fully-qualified non-deprecated name. It is also possible to use ```bash lake exe update_deprecations --mods One.Two.Three,Dd.Ee.Ff ``` to limit the scope of the replacements to the modules `One.Two.Three` and `Dd.Ee.Ff`. This is intended to be a first step in automating updates: combining this with a linter that emits appropriate warnings, the functionality of `lake exe update_deprecations` can be extended to perform more complicated updates. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta delegated awaiting-author 306/0 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/UpdateDeprecations.lean,MathlibTest/UpdateDeprecations.lean,lakefile.lean,scripts/README.md,scripts/update_deprecations.lean 7 15 ['YaelDillies', 'adomani', 'github-actions', 'j-loreaux', 'jcommelin', 'mathlib-bors', 'sgouezel'] joneugster
assignee:joneugster
150-14048
4 months ago
150-14048
4 months ago
34-82472
34 days
19378 adamtopaz
author:adamtopaz
feat: Explanation widgets This adds some simple widgets, wrapped in a tactic, term and command elaborator, for displaying markdown explanations in the infoview. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta awaiting-author 101/0 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Widget/Explain.lean 3 8 ['adamtopaz', 'eric-wieser', 'github-actions', 'joneugster', 'kmill'] nobody
149-16025
4 months ago
149-16025
4 months ago
49-80804
49 days
19323 madvorak
author:madvorak
feat: Function to Sum decomposition --- Discussion: https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Function.20to.20Sum.20decomposition t-data WIP 50/0 Mathlib.lean,Mathlib/Data/Sum/Decompose.lean 2 2 ['github-actions', 'madvorak'] nobody
147-22687
4 months ago
157-25285
5 months ago
43-18005
43 days
18461 hannahfechtner
author:hannahfechtner
feat: left and right common multiples mixins add mixins for left and right common multiples. These carry the data of what factors are used to create the common multiples --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra awaiting-author
label:t-algebra$
78/0 Mathlib/Algebra/Group/Defs.lean 1 13 ['github-actions', 'hannahfechtner', 'jcommelin', 'kbuzzard', 'kim-em', 'trivial1711'] nobody
140-38439
4 months ago
140-38439
4 months ago
69-35596
69 days
20797 vbeffara
author:vbeffara
feat(Topology/Covering): CM version of eq_of_comp_eq Add equivalents of the lemmas `IsCoveringMap.eq_of_comp_eq` and `IsCoveringMap.const_of_comp_CM` for the case of bundled `ContinuousMap` parameters. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-topology easy awaiting-author 9/1 Mathlib/Topology/Covering.lean 1 4 ['github-actions', 'ocfnash', 'vbeffara'] nobody
140-25204
4 months ago
141-26157
4 months ago
2-77310
2 days
13973 digama0
author:digama0
feat: lake exe refactor, initial framework This is the initial framework code for `lake exe refactor`. To use it, you add your refactoring to `Refactor/Main.lean` (note, you have to actually write some metaprogramming code here for the refactoring itself), and the harness will run it on specified files and apply the generated edits. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta awaiting-author 139/0 Refactor/Main.lean,lakefile.lean 2 10 ['adomani', 'digama0', 'eric-wieser', 'github-actions', 'joneugster', 'mattrobball'] nobody
137-16064
4 months ago
299-22391
9 months ago
4-80741
4 days
17589 joelriou
author:joelriou
feat(Algebra/ModuleCat/Presheaf): composition of pushforwards and pullbacks and compatibilites The composition of two pullback functors on presheaves of modules `pullback φ ⋙ pullback ψ` identifies to the pullback of the composition. We show compatibilites for these isomorphisms: they are deduced from similar identifies for pushforward (in which case they are `rfl`). --- - [x] depends on: #17366 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebraic-geometry t-category-theory WIP 166/2 Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Presheaf/Limits.lean,Mathlib/Algebra/Category/ModuleCat/Presheaf/Pullback.lean,Mathlib/Algebra/Category/ModuleCat/Presheaf/Pushforward.lean 4 4 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
137-5870
4 months ago
137-5889
4 months ago
0-0
0 seconds
21009 vihdzp
author:vihdzp
feat(Logic/Relation): more `TransGen` lemmas --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-logic t-order awaiting-author 13/0 Mathlib/Logic/Relation.lean 1 2 ['b-mehta', 'github-actions'] nobody
136-20842
4 months ago
136-20842
4 months ago
0-39342
10 hours
21035 mattrobball
author:mattrobball
draft --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
3/3 Mathlib/RingTheory/Kaehler/JacobiZariski.lean 1 4 ['github-actions', 'leanprover-bot', 'mattrobball'] nobody
135-77782
4 months ago
135-79621
4 months ago
0-0
0 seconds
15443 YaelDillies
author:YaelDillies
feat: The Marcinkiewicz-Zygmund inequality Prove the Marcinkiewicz-Zygmund inequality. The Marcinkiewicz-Zygmund inequality states that, if `X₁, ... Xₐ ∈ L^p` are independent random variables of mean zero valued in some inner product space, then the `L^p`-norm of `X₁ + ... + Xₐ` is at most `Cₚ` times the `L^(p/2)`-norm of `|X₁|² + ... + |Xₐ|²`, where `Cₚ` is a constant depending on `p` alone. From LeanAPAP Co-authored-by: Bhavik Mehta --- - [x] depends on: #15832 - [x] depends on: #21033 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis WIP 189/0 Mathlib.lean,Mathlib/Probability/MarcinkiewiczZygmund.lean 2 39 ['Parcly-Taxel', 'YaelDillies', 'b-mehta', 'github-actions', 'hrmacbeth', 'mathlib4-dependent-issues-bot', 'sgouezel'] nobody
135-39184
4 months ago
135-44248
4 months ago
89-28229
89 days
21039 eric-wieser
author:eric-wieser
hack: override `instance` to insert `fast_instance%` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta please-adopt 40/4 Mathlib/Algebra/Equiv/TransferInstance.lean,Mathlib/RingTheory/Ideal/Maximal.lean,Mathlib/Tactic/FastInstance.lean,Mathlib/Topology/FiberBundle/Basic.lean 4 1 ['github-actions'] nobody
135-18251
4 months ago
135-18251
4 months ago
0-0
0 seconds
20466 MohanadAhmed
author:MohanadAhmed
feat: Sherman Morrison formula for rank 1 update of the matrix inverse Provides the Sherman Morrison rank 1 update of the matrix inverse https://en.wikipedia.org/wiki/Sherman%E2%80%93Morrison_formula. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data awaiting-author 37/0 Mathlib/Data/Matrix/Invertible.lean 1 4 ['eric-wieser', 'github-actions'] nobody
133-18707
4 months ago
133-18707
4 months ago
23-30991
23 days
18749 GabinKolly
author:GabinKolly
feat(ModelTheory): preparatory work for the existence of Fraïsse limits Define the map of a PartialEquiv through an embedding, and related properties. Define embeddings and equivalences between equal structures or equal substructures, and related properties. Add miscellaneous lemmas which will be used to prove the existence of fraisse limits. --- This is preparation for #18876 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-logic awaiting-author 308/5 Mathlib/ModelTheory/Bundled.lean,Mathlib/ModelTheory/DirectLimit.lean,Mathlib/ModelTheory/FinitelyGenerated.lean,Mathlib/ModelTheory/PartialEquiv.lean,Mathlib/ModelTheory/Substructures.lean 5 9 ['GabinKolly', 'YaelDillies', 'github-actions', 'vihdzp'] nobody
129-81564
4 months ago
140-7618
4 months ago
73-63475
73 days
21277 GabinKolly
author:GabinKolly
feat(ModelTheory/PartialEquiv): Define the mapping of a self-partialEquiv through an embedding Define the mapping of a self-partialEquiv through an embedding and the notion of fully extendable partialEquiv. --- This is some preparatory work for #18876 - [ ] depends on: #21276 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-logic blocked-by-other-PR 215/5 Mathlib/ModelTheory/PartialEquiv.lean,Mathlib/ModelTheory/Substructures.lean 2 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
129-81288
4 months ago
129-81290
4 months ago
0-668
11 minutes
20649 GabinKolly
author:GabinKolly
feat(ModelTheory/Graph): prove characterization of the fraisse limit of finite simple graphs Prove that a countable graph with the extension property must be the Fraisse limit of finite simple graphs. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-logic t-combinatorics WIP 175/0 Mathlib/ModelTheory/Graph.lean,Mathlib/ModelTheory/Substructures.lean 2 1 ['github-actions'] nobody
127-77423
4 months ago
149-75064
4 months ago
0-0
0 seconds
19632 edegeltje
author:edegeltje
WIP CI --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) CI WIP 103/0 .github/workflows/on_pr_comment.yaml 1 1 ['github-actions'] nobody
127-21293
4 months ago
127-21293
4 months ago
0-0
0 seconds
21384 alreadydone
author:alreadydone
experiment: make submodule quotient reducibly defeq to additive group quotient --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
1/1 Mathlib/LinearAlgebra/Quotient/Defs.lean 1 1 ['github-actions'] nobody
126-9606
4 months ago
126-9609
4 months ago
0-0
0 seconds
10660 eric-wieser
author:eric-wieser
feat(LinearAlgebra/CliffordAlgebra): construction from a basis This is adapted from https://github.com/eric-wieser/lftcm2023-clifford_algebra, which only worked for the special case of `Q = 0`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra awaiting-author WIP
label:t-algebra$
573/0 Mathlib.lean,Mathlib/LinearAlgebra/CliffordAlgebra/Basis.lean 2 15 ['github-actions'] nobody
124-55644
4 months ago
124-55644
4 months ago
0-0
0 seconds
21450 eric-wieser
author:eric-wieser
feat: improve trace nodes for `positivity` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta 25/7 Mathlib/Tactic/Positivity/Core.lean 1 1 ['github-actions'] nobody
124-48975
4 months ago
124-48977
4 months ago
0-0
0 seconds
15355 adomani
author:adomani
feat: MiM PR report --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP 153/0 .github/workflows/monthly_pr_report.yaml,scripts/find_labels.sh 2 n/a ['YaelDillies', 'adomani', 'github-actions'] nobody
123-35566
4 months ago
unknown
unknown
21495 alreadydone
author:alreadydone
experiment: reducible HasQuotient.quotient' --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) bench-after-CI WIP 2/0 Mathlib/Algebra/Quotient.lean 1 1 ['github-actions'] nobody
123-29656
4 months ago
123-29656
4 months ago
0-200
3 minutes
21496 alreadydone
author:alreadydone
experiment: make SetLike.coe reducible --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) bench-after-CI t-data 1/1 Mathlib/Data/SetLike/Basic.lean 1 1 ['github-actions'] nobody
123-29425
4 months ago
123-29425
4 months ago
0-0
0 seconds
21447 erdOne
author:erdOne
feat(AlgebraicGeometry): the split algebraic torus --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebraic-geometry awaiting-author 419/0 Mathlib.lean,Mathlib/AlgebraicGeometry/Torus.lean 2 4 ['erdOne', 'github-actions', 'joelriou'] nobody
121-62830
4 months ago
121-81004
4 months ago
2-69252
2 days
21662 erdOne
author:erdOne
WIP: Weierstrass elliptic functions --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis 1595/0 Mathlib/Analysis/Elliptic/Basic.lean 1 1 ['github-actions'] nobody
119-17922
3 months ago
119-17923
3 months ago
0-0
0 seconds
19582 yu-yama
author:yu-yama
feat(GroupExtension/Abelian): define `OfMulDistribMulAction.equivH2` Mainly defines: - `structure GroupExtension.OfMulDistribMulAction N G [MulDistribMulAction G N]`: group extensions of `G` by `N` where the multiplicative action of `G` on `N` is the conjugation - `structure GroupExtension.OfMulDistribMulActionWithSection N G [MulDistribMulAction G N]`: group extensions with specific choices of sections - `def GroupExtension.OfMulDistribMulAction.equivH2`: a bijection between the equivalence classes of group extensions and $H^2 (G, N)$ - [x] depends on: #20802 (split PR: contains changes to the `Defs` file) - [x] depends on: #20998 (split PR: mainly adds the `Basic` file) - [ ] depends on: #21837 (split PR: adds the first part of the `Abelian` file) --- Here is a relevant TODO in Mathlib: https://github.com/leanprover-community/mathlib4/blob/4e9fa40d7c480937e09cd6e47a591bd6f3b8be42/Mathlib/RepresentationTheory/GroupCohomology/LowDegree.lean#L46-L48 I would appreciate your comments. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra blocked-by-other-PR
label:t-algebra$
736/14 Mathlib.lean,Mathlib/GroupTheory/GroupExtension/Abelian.lean,Mathlib/GroupTheory/GroupExtension/Defs.lean,docs/references.bib 4 3 ['erdOne', 'github-actions', 'mathlib4-dependent-issues-bot'] nobody
116-3145
3 months ago
116-6919
3 months ago
43-23183
43 days
20722 ctchou
author:ctchou
feat(Counterexamples): the Vitali set is non-measurable --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-measure-probability please-adopt awaiting-author 258/3 Counterexamples.lean,Counterexamples/VitaliSetNotMeasurable.lean,Mathlib/MeasureTheory/Measure/NullMeasurable.lean,docs/1000.yaml 4 74 ['ctchou', 'github-actions', 'grunweg', 'vihdzp'] vihdzp
assignee:vihdzp
115-80628
3 months ago
137-66236
4 months ago
0-0
0 seconds
20784 eric-wieser
author:eric-wieser
fix: prevent `exact?` recursing forever on `n = 55` Test case thanks to @llllvvuu: ```lean import Mathlib.SetTheory.Ordinal.Basic theorem natCast_inj {m n : ℕ} : (m : Ordinal) = n ↔ m = n := sorry example (n : Nat) : n = 55 := by exact? ``` This is surely a workaround for some unreported lean bug. The bug still exists for `n = 71` or higher, so we can still track down the bug after merging this patch. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-set-theory awaiting-author 22/3 Mathlib/SetTheory/Ordinal/Basic.lean,MathlibTest/LibrarySearchRecDepth.lean 2 12 ['Command-Master', 'eric-wieser', 'github-actions', 'kbuzzard', 'kim-em', 'leanprover-bot', 'mattrobball'] nobody
111-84499
3 months ago
111-84499
3 months ago
32-73698
32 days
22037 EtienneC30
author:EtienneC30
issues with Finset subtype coercion [Zulip discussion](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Finset.20subtype.20changes) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data 7/1 Mathlib/Data/Finset/Defs.lean,Mathlib/MeasureTheory/Constructions/Projective.lean 2 1 ['github-actions'] nobody
111-34453
3 months ago
111-34505
3 months ago
0-0
0 seconds
22092 fpvandoorn
author:fpvandoorn
perf: lower gcongr priority in group mono lemmas --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra WIP
label:t-algebra$
13/9 Mathlib/Algebra/Order/Monoid/Unbundled/Basic.lean 1 5 ['fpvandoorn', 'github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot'] nobody
110-4536
3 months ago
110-4621
3 months ago
0-6118
1 hour
13442 dignissimus
author:dignissimus
feat: mabel tactic for multiplicative abelian groups Mabel tactic for multiplicative abelian groups (#10361) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-meta modifies-tactic-syntax awaiting-author help-wanted 439/0 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/MAbel.lean,MathlibTest/mabel.lean 4 10 ['BoltonBailey', 'dignissimus', 'github-actions', 'joneugster', 'kbuzzard'] joneugster
assignee:joneugster
109-77367
3 months ago
114-58963
3 months ago
0-16
16 seconds
21501 sksgurdldi
author:sksgurdldi
feat(List): add sum_zipWith_eq_finset_sum ### **Description:** This PR adds the lemma `List.sum_zipWith_eq_finset_sum` to `Mathlib.Algebra.BigOperators.Group.Finset.Basic`. #### **Statement:** The sum of the `zipWith` operation on two lists equals the sum of applying the operation to corresponding elements of the two lists, indexed over the minimum of their lengths. #### **Formal Statement:** ```lean lemma sum_zipWith_eq_finset_sum [Inhabited α] [Inhabited β] [AddCommMonoid γ] {op : α → β → γ} (l : List α) (m : List β) : (List.zipWith op l m).sum = ∑ x ∈ (Finset.range (Nat.min l.length m.length)), op (l[x]!) (m[x]!) ``` #### **Remarks:** - This lemma provides a useful equivalence between `List.zipWith` and summation over a `Finset.range` indexed by `Nat.min l.length m.length`. - It can be helpful in algebraic manipulations involving list-based summations. #### **Dependencies:** No additional dependencies. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra awaiting-author
label:t-algebra$
43/0 Mathlib/Algebra/BigOperators/Group/Finset/Basic.lean 1 1 ['github-actions', 'j-loreaux'] nobody
109-76446
3 months ago
109-76446
3 months ago
13-33168
13 days
20956 tomaz1502
author:tomaz1502
feat(Computability/QueryComplexity/Sort.lean): Formalization of upper bound of queries for merge sort This PR builds on top of #20924 to prove that merge sort (as defined in Lean's library) never executes more than `3 * n * ceil_log2 n` comparisons, where `n` is the size of the input list and `ceil_log2` is the ceil of the logarithm in base 2, which is defined in this PR. Zulip discussion: https://leanprover.zulipchat.com/#narrow/channel/144837-PR-reviews/topic/.2318629.20runtime.20complexity.20of.20sorting.20a.20list - [ ] depends on: #20924 Co-authored-by: Geoffrey Irving --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-computability blocked-by-other-PR 676/0 Mathlib.lean,Mathlib/Computability/QueryComplexity/Basic.lean,Mathlib/Computability/QueryComplexity/Defs.lean,Mathlib/Computability/QueryComplexity/Sort.lean 4 3 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
108-86364
3 months ago
138-13477
4 months ago
0-41
41 seconds
22194 eric-wieser
author:eric-wieser
feat: oracle computations (alternative) This explores a simpler version of #20924 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-computability 698/0 Archive/Examples/SumOracle.lean,Mathlib.lean,Mathlib/Computability/QueryComplexity/Defs.lean,Mathlib/Computability/QueryComplexity/Sort.lean 4 4 ['eric-wieser', 'girving', 'github-actions'] nobody
106-31303
3 months ago
106-72191
3 months ago
0-0
0 seconds
22233 pechersky
author:pechersky
feat(Algebra/Valued): `AdicExpansion.evalAt` --- - [ ] depends on: #22231 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology blocked-by-other-PR 488/0 Mathlib.lean,Mathlib/Topology/Algebra/Valued/AdicExpansion.lean 2 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
105-61062
3 months ago
105-61064
3 months ago
0-412
6 minutes
22232 pechersky
author:pechersky
feat(Algebra/Valued): `AdicExpansion.apprUpto` --- - [ ] depends on: #22231 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology blocked-by-other-PR 399/0 Mathlib.lean,Mathlib/Topology/Algebra/Valued/AdicExpansion.lean 2 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
105-61060
3 months ago
105-61063
3 months ago
0-414
6 minutes
18230 digama0
author:digama0
feat(Tactic/ScopedNS): extend `scoped[NS]` to more commands refactor `ScopedNS` to remove error prone repetitiveness and extend it to other commands such as `syntax`, `macro`, `elab`, etc. Co-authored-by: Jon Eugster --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta awaiting-author 194/26 Mathlib/Tactic/ScopedNS.lean,MathlibTest/scopedNS.lean 2 6 ['adomani', 'digama0', 'github-actions', 'joneugster', 'kbuzzard'] nobody
105-32905
3 months ago
105-32905
3 months ago
41-32344
41 days
19062 hannahfechtner
author:hannahfechtner
feat(Algebra/PresentedMonoid/Basic) : facts about rel Add in a number of useful theorems (reflexivity, closure under multiplication) and lemmas about when the PresentedMonoid.rel holds as an API for users --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra awaiting-author
label:t-algebra$
38/0 Mathlib/GroupTheory/Congruence/Defs.lean 1 8 ['github-actions', 'hannahfechtner', 'kbuzzard', 'riccardobrasca'] nobody
104-27615
3 months ago
104-27615
3 months ago
87-64575
87 days
22302 CharredLee
author:CharredLee
feat: add `CategoryTheory.Topos.Power` This is a continuation of #21281 with the end goal of defining topoi in Mathlib. It introduces the notion of a power object in a category with a subobject classifier, which is a special case of an internal hom. The definition `HasPowerObjects C` contained in this PR is all that remains before `IsTopos C` can be defined. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-category-theory awaiting-author 312/0 Mathlib.lean,Mathlib/CategoryTheory/Topos/Power.lean 2 2 ['github-actions', 'joelriou'] b-mehta
assignee:b-mehta
103-77642
3 months ago
103-78769
3 months ago
0-1528
25 minutes
22330 jjdishere
author:jjdishere
feat(RingTheory/Perfection): lemmas for `frobeniusEquiv.symm` In this PR, we add several simp lemmas for `frobeniusEquiv.symm` and `frobeniusEquiv.symm^[n]`. We also modified `ModP` from a definition to an abbreviation to make the `Ideal.Quotient` APIs work on `ModP`. #21564 depends on this PR. --- - [ ] depends on: #22320 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra blocked-by-other-PR
label:t-algebra$
321/5 Mathlib.lean,Mathlib/Algebra/Ring/Aut.lean,Mathlib/FieldTheory/Perfect.lean,Mathlib/RingTheory/Perfection.lean,Mathlib/RingTheory/Perfectoid/Untilt.lean,Mathlib/RingTheory/WittVector/Basic.lean,Mathlib/RingTheory/WittVector/Complete.lean,Mathlib/RingTheory/WittVector/TeichmullerSeries.lean 8 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
103-15599
3 months ago
103-15601
3 months ago
0-822
13 minutes
21915 YaelDillies
author:YaelDillies
feat: simproc for `Int.divisorsAntidiag` Co-authored-by: Paul Lezeau --- - [x] depends on: #21912 - [x] depends on: #21991 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta WIP 73/0 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Simproc/DivisorsAntidiag.lean 3 7 ['YaelDillies', 'eric-wieser', 'github-actions', 'mathlib4-dependent-issues-bot'] nobody
101-18302
3 months ago
101-18317
3 months ago
0-260
4 minutes
22416 JLimperg
author:JLimperg
chore: fix benchmark script for precompilation The benchmarking script used to fail when precompilation was enabled anywhere in the dependency graph. --- Fix courtesy of @Kha. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 2/0 scripts/bench/fake-root/lib/lean/libleanshared.so,scripts/bench/run 2 1 ['github-actions'] nobody
100-73697
3 months ago
100-73760
3 months ago
0-0
0 seconds
22389 adomani
author:adomani
feat: the variableVariable linter The motivation comes from [this Zulip discussion](https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/style.20proposal.3A.20avoid.20.60variable.20.7BX.7D.20.2E.2E.2E.20variable.20.28X.29.60). Summarising, updating a variable binder for a single declaration can be confusing. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-linter WIP 167/0 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter.lean,Mathlib/Tactic/Linter/VariableVariable.lean,variableDeclarationVariable_replacements.py 5 1 ['github-actions'] nobody
99-14764
3 months ago
101-35920
3 months ago
0-0
0 seconds
22390 YunkaiZhang233
author:YunkaiZhang233
feat(CategoryTheory): implemented proofs for factorisation categories being equivalent to iterated comma categories in two ways Completed one of the tasks in TODOs, shown and implemented the details for `(X/C)/f ≌ Factorisation f ≌ f/(C/Y)`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-category-theory awaiting-author 112/1 Mathlib/CategoryTheory/Category/Factorisation.lean 1 9 ['YunkaiZhang233', 'github-actions', 'joelriou'] nobody
98-31875
3 months ago
101-27347
3 months ago
0-6513
1 hour
22320 jjdishere
author:jjdishere
feat(RingTheory/WittVector): the Teichmuller series In this PR, we show that every element `x` of the Witt vectors `𝕎 R` can be written as the (`p`-adic) summation of the Teichmuller series. Instead of using `tsum`, we only show that `p ^ (n + 1)` divides `x` minus the summation of the first `n + 1` terms of the Teichmuller series. We also show that if `p` divides the first (n + 1) coefficients of a Witt vector, then `p^(n+1)` divides the `n`-th ghost component. #21564 depends on this PR. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra awaiting-author
label:t-algebra$
204/2 Mathlib.lean,Mathlib/Algebra/Ring/Aut.lean,Mathlib/FieldTheory/Perfect.lean,Mathlib/RingTheory/WittVector/Basic.lean,Mathlib/RingTheory/WittVector/Complete.lean,Mathlib/RingTheory/WittVector/TeichmullerSeries.lean 6 12 ['github-actions', 'jjdishere', 'riccardobrasca'] nobody
97-25322
3 months ago
97-25322
3 months ago
6-3646
6 days
22497 adomani
author:adomani
test: decl diff in lean Testing branch for #22464. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) test-ci CI WIP 161/0 .github/workflows/PR_summary_lean.yml,Mathlib.lean,Mathlib/Test.lean,scripts/README.md,scripts/declarations_diff.lean,scripts/declarations_diff_lean_shell_glue.sh 6 7 ['github-actions', 'mergify'] nobody
97-14342
3 months ago
98-26041
3 months ago
0-0
0 seconds
20636 eric-wieser
author:eric-wieser
feat: multiplication of intervals in rings --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra awaiting-author
label:t-algebra$
36/1 Mathlib/Algebra/Order/Interval/Basic.lean 1 16 ['Timeroot', 'YaelDillies', 'eric-wieser', 'github-actions'] nobody
97-2963
3 months ago
133-6740
4 months ago
17-17852
17 days
16000 YaelDillies
author:YaelDillies
feat: Croot-Sisask Almost Periodicity Almost periodicity is nowadays a standard tool in additive combinatorics. From LeanAPAP --- - [ ] depends on: #15443 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis t-combinatorics blocked-by-other-PR 0/0 0 4 ['github-actions', 'leanprover-community-mathlib4-bot', 'mergify'] nobody
96-32284
3 months ago
96-32289
3 months ago
0-159
2 minutes
22642 grunweg
author:grunweg
WIP: add `mfderiv_prod` and `mfderiv_prodMap` Help with these sorries is very welcome! Part of my bordism theory project: these will be needed for #22059. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-differential-geometry WIP 27/0 Mathlib/Geometry/Manifold/MFDeriv/SpecificFunctions.lean 1 1 ['github-actions'] nobody
95-21116
3 months ago
95-21116
3 months ago
0-8
8 seconds
22648 adomani
author:adomani
test: lean implementation decl diff quandle --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 210/1 .github/workflows/PR_summary_lean.yml,Mathlib/Algebra/Quandle.lean,scripts/README.md,scripts/declarations_diff.lean,scripts/declarations_diff_lean_shell_glue.sh 5 4 ['adomani', 'eric-wieser', 'github-actions'] nobody
93-45122
3 months ago
95-14408
3 months ago
0-0
0 seconds
22741 joelriou
author:joelriou
feat(CategoryTheory/Abelian/SerreClass): left Bousfield localizations If `G : D ⥤ C` is an exact functor between abelian categories, with a fully faithful right adjoint `F`, then `G` identifies `C` to the localization of `D` with respect to the class of morphisms `G.kernel.isoModSerre`, i.e. `D` is the localization of `C` with respect to Serre class `G.kernel` consisting of the objects in `D` that are sent to a zero object by `G`. (We also translate this in terms of a left Bousfield localization.) --- - [ ] depends on: #22739 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory blocked-by-other-PR 263/0 Mathlib.lean,Mathlib/CategoryTheory/Abelian/SerreClass/Bousfield.lean,Mathlib/CategoryTheory/Abelian/SerreClass/MorphismProperty.lean,Mathlib/CategoryTheory/Limits/Shapes/Equalizers.lean,Mathlib/CategoryTheory/Limits/Shapes/Kernels.lean,Mathlib/CategoryTheory/ObjectProperty/ContainsZero.lean 6 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
91-40449
2 months ago
92-11082
3 months ago
0-1246
20 minutes
10084 alreadydone
author:alreadydone
draft for Van Kampen The part about the homotopy lifting property for covering maps has been extracted to #22649 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology WIP 91/24 Mathlib/AlgebraicTopology/FundamentalGroupoid/Basic.lean,Mathlib/AlgebraicTopology/FundamentalGroupoid/VanKampen.lean 2 0 [] nobody
91-17426
2 months ago
498-2809
1 year ago
0-0
0 seconds
22784 grunweg
author:grunweg
feat: add Diffeomorph.sumSumSumComm This matches `{Equiv,Homeomorph.sumSumSumComm}`, and is needed to prove that addition in the cobordism group is commutatives. From my bordism theory project. --- - depends on #22783 (easy pre-requisites) The current proof is not complete yet, and feels very painful. I'm not yet sure what's the best way to write this. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-differential-geometry WIP 50/0 Mathlib/Geometry/Manifold/Diffeomorph.lean 1 1 ['github-actions'] nobody
90-85195
2 months ago
91-21539
2 months ago
0-0
0 seconds
22820 chrisflav
author:chrisflav
chore: fix `Scheme.Hom.appTop` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebraic-geometry 67/35 Mathlib/AlgebraicGeometry/AffineScheme.lean,Mathlib/AlgebraicGeometry/GammaSpecAdjunction.lean,Mathlib/AlgebraicGeometry/Restrict.lean,Mathlib/AlgebraicGeometry/Scheme.lean 4 1 ['github-actions'] nobody
90-40805
2 months ago
90-40807
2 months ago
0-0
0 seconds
22846 mattrobball
author:mattrobball
test t-analysis 2/0 Mathlib/Analysis/Normed/Module/Basic.lean 1 4 ['github-actions', 'leanprover-bot', 'mattrobball'] nobody
90-3303
2 months ago
90-5243
2 months ago
0-0
0 seconds
22749 joelriou
author:joelriou
feat(CategoryTheory/Abelian): the Gabriel-Popescu theorem as a localization with respect to a Serre class This PR introduces a structure `GabrielPopescuPackage C` which contains the information to say that the abelian category `C` is a localization of a category of modules with respect to a suitable Serre class. --- - [ ] depends on: #22739 - [ ] depends on: #22741 - [x] depends on: #22733 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory blocked-by-other-PR 376/4 Mathlib.lean,Mathlib/CategoryTheory/Abelian/GrothendieckCategory/ModuleEmbedding/GabrielPopescu.lean,Mathlib/CategoryTheory/Abelian/SerreClass/Bousfield.lean,Mathlib/CategoryTheory/Abelian/SerreClass/MorphismProperty.lean,Mathlib/CategoryTheory/Limits/Shapes/Equalizers.lean,Mathlib/CategoryTheory/Limits/Shapes/Kernels.lean,Mathlib/CategoryTheory/ObjectProperty/ContainsZero.lean 7 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
88-86122
2 months ago
88-86137
2 months ago
0-2391
39 minutes
22928 javra
author:javra
feat(CategoryTheory): infrastructure for inclusion morphisms into products in categories with 0-morphisms --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory 52/14 Mathlib/CategoryTheory/Limits/Shapes/BinaryBiproducts.lean,Mathlib/CategoryTheory/Limits/Shapes/Biproducts.lean,Mathlib/CategoryTheory/Limits/Shapes/ZeroMorphisms.lean 3 1 ['github-actions'] nobody
87-22934
2 months ago
87-23115
2 months ago
87-23157
87 days
22952 eric-wieser
author:eric-wieser
refactor: reimplement `RingQuot` in terms of `RingCon.Quotient` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
157/184 Mathlib/Algebra/RingQuot.lean,Mathlib/GroupTheory/Congruence/Basic.lean,Mathlib/RingTheory/Congruence/Basic.lean,Mathlib/RingTheory/Congruence/Defs.lean 4 1 ['github-actions'] nobody
86-28245
2 months ago
86-28245
2 months ago
0-0
0 seconds
22159 shetzl
author:shetzl
feat: add definition of pushdown automata Add the definition of pushdown automata and their two acceptance conditions: acceptance based on empty stack and acceptance based on final state. Co-authored-by: Tobias Leichtfried --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-computability new-contributor awaiting-author 70/0 Mathlib.lean,Mathlib/Computability/PDA.lean 2 34 ['YaelDillies', 'github-actions', 'madvorak', 'shetzl'] nobody
84-38789
2 months ago
84-38789
2 months ago
20-81771
20 days
23042 joneugster
author:joneugster
feat(CategoryTheory/Enriched/Limits): add HasConicalLimitsOfSize.shrink --- Note: I've marked this "WIP" because I'm not yet sure when this will be needed and I'd probably put the PR on the queue once I've created some follow-up needing it. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) infinity-cosmos t-category-theory WIP 22/1 Mathlib/CategoryTheory/Enriched/Limits/HasConicalLimits.lean 1 1 ['github-actions'] nobody
83-36901
2 months ago
83-37056
2 months ago
0-1
1 second
17587 kmill
author:kmill
feat: Sym2-as-Finset theory --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data new-contributor 105/3 Mathlib/Combinatorics/SimpleGraph/Basic.lean,Mathlib/Combinatorics/SimpleGraph/Finite.lean,Mathlib/Data/Sym/Sym2.lean,Mathlib/RingTheory/Polynomial/Vieta.lean 4 10 ['FordUniver', 'YaelDillies', 'github-actions', 'kmill'] nobody
82-49314
2 months ago
82-84794
2 months ago
0-0
0 seconds
18091 tukamilano
author:tukamilano
feat: Hoeffding's lemma Formalize Hoeffding's lemma using the property of cumulant. Co-authored-by: Yuma Mizuno [mizuno.y.aj@gmail.com](mailto:mizuno.y.aj@gmail.com) --- - [x] depends on: #20151 large-import new-contributor t-measure-probability awaiting-author 339/0 Mathlib.lean,Mathlib/Probability/Hoeffding.lean,Mathlib/Probability/Moments/Basic.lean,Mathlib/Probability/Moments/MGFAnalytic.lean,docs/references.bib 5 55 ['RemyDegenne', 'YaelDillies', 'github-actions', 'mathlib4-dependent-issues-bot', 'tukamilano', 'yuma-mizuno'] tukamilano
assignee:tukamilano
81-30405
2 months ago
81-30413
2 months ago
1-58489
1 day
16239 Rida-Hamadani
author:Rida-Hamadani
feat(Geometry/Manifold): orientable manifolds This module defines orientable manifolds. [This](https://leanprover.zulipchat.com/#narrow/stream/217875-Is-there-code-for-X.3F/topic/Orientable.20Surface) Zulip topic is related. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-differential-geometry awaiting-author 376/6 Mathlib.lean,Mathlib/Geometry/Manifold/Instances/Real.lean,Mathlib/Geometry/Manifold/Orientable.lean 3 39 ['Rida-Hamadani', 'github-actions', 'grunweg', 'ocfnash'] nobody
80-71961
2 months ago
100-24283
3 months ago
5-70530
5 days
23142 joneugster
author:joneugster
feat(CategoryTheory/Enriched/Limits): add API for HasConicalLimit --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) infinity-cosmos t-category-theory awaiting-author 52/9 Mathlib/CategoryTheory/Enriched/Limits/HasConicalLimits.lean 1 2 ['github-actions', 'joelriou'] nobody
80-40047
2 months ago
80-40047
2 months ago
0-68906
19 hours
23004 Vierkantor
author:Vierkantor
Benchmarking for #22950 This is a rebase of #22950 on top of the changes of #22907 so we can see the true difference in benchmarking. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data WIP 10/6 Mathlib/Data/Complex/Exponential.lean,Mathlib/Data/PFun.lean 2 10 ['Vierkantor', 'github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot'] nobody
78-77423
2 months ago
78-77423
2 months ago
0-0
0 seconds
19607 madvorak
author:madvorak
Block matrix totally unimodular --- Discussion: https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/TU.20block.20matrix.20.2319607 - [ ] depends on: #19323 - [ ] depends on: #20428 - [ ] depends on: #20433 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR WIP 156/0 Mathlib.lean,Mathlib/Data/Sum/Decompose.lean,Mathlib/LinearAlgebra/Matrix/Determinant/TotallyUnimodular.lean 3 10 ['github-actions', 'jcommelin', 'madvorak', 'mathlib4-dependent-issues-bot'] nobody
77-12122
2 months ago
77-12122
2 months ago
0-0
0 seconds
23285 AntoineChambert-Loir
author:AntoineChambert-Loir
refactor: directed systems in terms of functors This is a WIP aiming to refactor the work on directed systems using the category theory library. But there are universes nightmares. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-algebra t-category-theory WIP
label:t-algebra$
111/45 Mathlib/Order/DirectedInverseSystem.lean 1 1 ['github-actions'] nobody
76-76838
2 months ago
76-76844
2 months ago
0-24
24 seconds
9820 jjaassoonn
author:jjaassoonn
feat(RingTheory/GradedAlgebra/HomogeneousIdeal): generalize to homogeneous submodule The definitions, constructions and theorems in `HomogeneousIdeal.lean` are generalized to a homogeneous submodules. So say $R$ is a ring and $M \cong \bigoplus_{i} M_i$ is an $R$-module. Then a homogeneous $R$-submodule of $M$ is an $R$-submodule $N$ such that for all $i$ and $n \in N$, $n_i \in N$. Note that this notion doesn't actually require $R$ to be graded and $M$ is a graded module. But for more interesting lemmas, we do need that $M$ is graded $R$-module. We bake the fact $R$ is graded into the definition of homogeneous submodule, otherwise, `CompleteLattice HomogeneousSubmodule` cannot find the order of synthesis (the proof depends on that $R$ is graded) All definitions/constructions/theorems have a copy for ideals as well, this is to make sure dot notation still works. The motivation of this generalization is graded quotient module --- - [ ] depends on:#18728 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
515/185 Mathlib/Algebra/Module/GradedModule.lean,Mathlib/AlgebraicGeometry/ProjectiveSpectrum/Scheme.lean,Mathlib/RingTheory/GradedAlgebra/Homogeneous/Ideal.lean,Mathlib/RingTheory/GradedAlgebra/Homogeneous/Submodule.lean,scripts/nolints_prime_decls.txt 5 2 ['github-actions'] nobody
74-8833
2 months ago
116-67285
3 months ago
147-32024
147 days
21344 kbuzzard
author:kbuzzard
chore: attempt to avoid diamond in OreLocalization --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra awaiting-author
label:t-algebra$
16/5 Mathlib/RingTheory/OreLocalization/Basic.lean 1 5 ['erdOne', 'github-actions', 'kbuzzard'] nobody
74-6543
2 months ago
74-6543
2 months ago
53-20069
53 days
23460 Timeroot
author:Timeroot
feat: Definition of `Clone` Basics about Clones. Part of #20051 --- - [ ] depends on: #23459 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra blocked-by-other-PR
label:t-algebra$
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
71-1930
2 months ago
71-1930
2 months ago
0-1312
21 minutes
21693 erdOne
author:erdOne
feat: taylor expansion of `1 / z ^ r` --- This might exist somewhere else but I couldn't find them. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis awaiting-author 96/0 Mathlib.lean,Mathlib/Analysis/SpecificLimits/InvPow.lean 2 10 ['erdOne', 'eric-wieser', 'github-actions', 'j-loreaux'] nobody
70-66429
2 months ago
115-19500
3 months ago
3-59857
3 days
21837 yu-yama
author:yu-yama
feat(GroupExtension/Abelian): define `conjClassesEquivH1` As the third part of #19582, this PR adds the first part of the `Abelian` file. It mainly: - defines `SemidirectProduct.conjClassesEquivH1`, a bijection between the conjugacy classes of splittings of a group extension associated to a semidirect product and $H^1 (G, N)$. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra awaiting-author
label:t-algebra$
129/3 Mathlib.lean,Mathlib/GroupTheory/GroupExtension/Abelian.lean,Mathlib/GroupTheory/GroupExtension/Defs.lean,docs/references.bib 4 4 ['erdOne', 'github-actions'] erdOne
assignee:erdOne
69-39888
2 months ago
69-39888
2 months ago
46-55213
46 days
22355 xyzw12345
author:xyzw12345
feat(Algebra/RingQuot): Some lemmas about `RingQuot.mkAlgHom` and `RingQuot.mkRingHom` This PR provides a few basic lemmas about `RingQuot.mkRingHom` and `RingQuot.mkAlgHom`. These lemmas are about when are two elements mapped to the same one under these two maps, and they correspond to the lemma `Quot.eq`. PR #22279 depends on these lemmas. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra awaiting-author
label:t-algebra$
16/0 Mathlib/Algebra/RingQuot.lean 1 13 ['Paul-Lez', 'erdOne', 'eric-wieser', 'github-actions', 'ocfnash', 'xyzw12345'] nobody
68-52022
2 months ago
69-39345
2 months ago
32-33842
32 days
21829 Whysoserioushah
author:Whysoserioushah
feat(LinearAlgebra/TensorProduct/HomTensor): Add TensorProduct of Hom-modules Co-authored-by: Andrew Yang --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra awaiting-author
label:t-algebra$
174/0 Mathlib.lean,Mathlib/LinearAlgebra/TensorProduct/HomTensor.lean 2 26 ['Whysoserioushah', 'YaelDillies', 'erdOne', 'github-actions', 'kbuzzard'] nobody
68-33061
2 months ago
69-39581
2 months ago
46-53384
46 days
6718 FR-vdash-bot
author:FR-vdash-bot
feat: Lindemann-Weierstrass Theorem --- There's still a lot of work to be done before it gets into mathlib. - [x] depends on: #6593 - [x] depends on: #6719 - [x] depends on: #6723 - [x] depends on: #6740 - [x] depends on: #7274 - [x] depends on: #8807 - [x] depends on: #12191 - [x] depends on: #12764 - [x] depends on: #16259 - [x] depends on: #16262 - [x] depends on: #16886 - [x] depends on: #16898 - [x] depends on: #16923 - [x] depends on: #16933 - [x] depends on: #17119 - [x] depends on: #17893 - [x] depends on: #17894 - [x] depends on: #17896 - [x] depends on: #18556 - [ ] depends on: #18693 - [x] depends on: #19225 - [x] depends on: #19246 - [x] depends on: #20092 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-analysis blocked-by-other-PR WIP
label:t-algebra$
1360/51 Mathlib.lean,Mathlib/Algebra/MonoidAlgebra/Basic.lean,Mathlib/FieldTheory/Minpoly/ConjRootClass.lean,Mathlib/FieldTheory/Minpoly/IsConjRoot.lean,Mathlib/NumberTheory/Transcendental/Lindemann/AlgebraicPart.lean,Mathlib/NumberTheory/Transcendental/Lindemann/AnalyticalPart.lean,Mathlib/NumberTheory/Transcendental/Lindemann/Basic.lean,Mathlib/NumberTheory/Transcendental/Lindemann/SumAEvalARoots.lean,Mathlib/RingTheory/MvPolynomial/Symmetric/Eval.lean,docs/100.yaml,docs/1000.yaml 11 n/a ['FR-vdash-bot', 'Ruben-VandeVelde', 'acmepjz', 'alreadydone', 'eric-wieser', 'github-actions', 'j-loreaux', 'jcommelin', 'jjdishere', 'mathlib4-dependent-issues-bot'] Ruben-VandeVelde
assignee:Ruben-VandeVelde
68-8190
2 months ago
unknown
unknown
22861 eric-wieser
author:eric-wieser
feat: add the trace of a bilinear form Following the steps at [#Is there code for X? > Laplacian @ 💬](https://leanprover.zulipchat.com/#narrow/channel/217875-Is-there-code-for-X.3F/topic/Laplacian/near/450834505). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) Some questions: * Does this generalize to multilinear maps? * Is there an `RCLike` generalization? * Does this generalize to `BilinMap` instead of just `BilinForm`? Perhaps the approach in [#mathlib4 > Stating Schrodinger's equation @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Stating.20Schrodinger's.20equation/near/500409890) of using `ContinuousLinearMap.adjoint'` is better. t-algebra awaiting-author
label:t-algebra$
100/0 Mathlib.lean,Mathlib/LinearAlgebra/BilinearForm/Trace.lean 2 3 ['github-actions', 'jcommelin'] nobody
66-22900
2 months ago
66-22900
2 months ago
23-44995
23 days
20330 mans0954
author:mans0954
feat(Analysis/Normed/Module/Complemented): The idempotent associated with a complemented subspace Given a complemented subspace `p` of a Banach space `E`, with complement `q`, there exists an idempotent `P` in the ring `E →L[𝕜] E` such that `P` has range `p` and kernel `q`. Similarly `1-P` has range `q` and kernel `p`. See Rudin, Functional Analysis, Theorem 5.16. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-analysis WIP 185/3 Mathlib/Algebra/Module/End.lean,Mathlib/Algebra/Module/Hom.lean,Mathlib/Algebra/Module/LinearMap/End.lean,Mathlib/Analysis/Normed/Module/Complemented.lean,Mathlib/RingTheory/Idempotents.lean 5 14 ['YaelDillies', 'alreadydone', 'github-actions', 'j-loreaux', 'kbuzzard', 'mans0954', 'urkud'] nobody
65-55617
2 months ago
119-3316
3 months ago
0-0
0 seconds
19969 mans0954
author:mans0954
WiP: Star Linear Maps and Star Submodules WiP: Star Linear Maps and Star Submodules --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra WIP
label:t-algebra$
1729/0 Mathlib.lean,Mathlib/Algebra/Star/StarLinearMap.lean,Mathlib/Algebra/Star/Submodule.lean 3 1 ['github-actions'] nobody
65-55522
2 months ago
176-80700
5 months ago
0-0
0 seconds
14369 mans0954
author:mans0954
feat(Analysis/NormedSpace/MStructure): M-ideals WiP: Define M-ideals and establish basic properties. --- - [x] depends on: #14458 - [ ] depends on : #20084 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-analysis WIP 857/40 Mathlib/Algebra/Module/End.lean,Mathlib/Algebra/Module/Hom.lean,Mathlib/Algebra/Module/LinearMap/End.lean,Mathlib/Analysis/Normed/Module/Complemented.lean,Mathlib/Analysis/NormedSpace/MStructure.lean 5 n/a ['github-actions', 'leanprover-community-mathlib4-bot'] nobody
65-55133
2 months ago
unknown
unknown
13918 mans0954
author:mans0954
feat(Topology/Order/HullKernel): Add the Hull-Kernel Topology Let `α` be a `CompleteLattice` and let `T` be a subset of `α`. The relative `Topology.lower` on `T` takes on a particularly simple form when every element of `T` is `InfPrime` in `α`. In this case, the relative-open sets are exactly the sets of the form `T ↓∩ (Ici a)ᶜ` for some `a` in `α`. The pair of maps `S → ⊓ S` and `a → T ↓∩ Ici a` are often referred to as the kernel and the hull. They form an antitone Galois connection between the subsets of `T` and `α`. When `α` can be generated from `T` by taking infs, this becomes a Galois insertion and the topological closure coincides with the closure arising from the Galois insertion. For this reason the relative lower topology on `T` is often referred to as the hull-kernel topology. The names Jacobson topology and structure topology also occur in the literature. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order t-topology awaiting-author 302/0 Mathlib.lean,Mathlib/Data/Set/Subset.lean,Mathlib/Topology/Order/HullKernel.lean,docs/references.bib 4 n/a ['YaelDillies', 'github-actions', 'mans0954'] nobody
65-55065
2 months ago
unknown
unknown
21814 mans0954
author:mans0954
feature(LinearAlgebra/QuadraticForm/TensorProduct): Extend `baseChange_ext` to work over a free module WiP: Extend `baseChange_ext` to work over a free module --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra WIP
label:t-algebra$
105/5 Mathlib/LinearAlgebra/Basis/Bilinear.lean,Mathlib/LinearAlgebra/QuadraticForm/TensorProduct.lean 2 1 ['github-actions'] nobody
63-49756
2 months ago
116-44398
3 months ago
0-0
0 seconds
18705 mans0954
author:mans0954
feat(Algebra/Module/NestAlgebra): Nest algebras Nest algebras are an operator analogue of upper triangular matrices. They have been extensively studied in the context of Hilbert spaces, but also in more general contexts. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order t-algebra awaiting-author
label:t-algebra$
184/0 Mathlib.lean,Mathlib/Algebra/Module/NestAlgebra.lean,Mathlib/Order/Nest.lean,Mathlib/Order/Preorder/Chain.lean,docs/references.bib 5 8 ['github-actions', 'j-loreaux', 'mans0954'] j-loreaux
assignee:j-loreaux
63-49444
2 months ago
63-49457
2 months ago
2-67791
2 days
19806 mans0954
author:mans0954
WiP: Expansion of the tensor product of quadratic maps over a linear combination WiP --- - [ ] depends on: #18578 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra WIP
label:t-algebra$
483/0 Mathlib/Data/Sym/Sym2/Prod.lean,Mathlib/LinearAlgebra/QuadraticForm/Basic.lean,Mathlib/LinearAlgebra/QuadraticForm/Basis.lean,Mathlib/LinearAlgebra/QuadraticForm/TensorProduct.lean 4 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
63-47351
2 months ago
63-49626
2 months ago
0-0
0 seconds
22888 plp127
author:plp127
perf: replace `Lean.Expr.swapBVars` with a better? implementation Replaces `Lean.Expr.swapBVars` with a version that traverses the expression. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta awaiting-author 14/12 Mathlib/Tactic/FunProp/ToBatteries.lean 1 23 ['eric-wieser', 'github-actions', 'joneugster', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'plp127'] eric-wieser and joneugster
assignee:eric-wieser assignee:joneugster
63-35146
2 months ago
64-21445
2 months ago
4-80306
4 days
18437 ADedecker
author:ADedecker
refactor: add refactored APIs for algebraic filter bases This is the first part of the refactor of algebraic filter bases discussed [here](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Refactoring.20algebraic.20filter.20bases/near/479437345). This adds the new APIs without touching any existing file in order to split the work. **Please review this by comparing with the existing API!** See #18202 for the full picture. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-topology awaiting-author
label:t-algebra$
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 21 ['ADedecker', 'AntoineChambert-Loir', 'eric-wieser', 'github-actions'] PatrickMassot
assignee:PatrickMassot
63-23856
2 months ago
135-53952
4 months ago
75-64682
75 days
23772 SEU-Prime
author:SEU-Prime
Create Amice.lean i built amice equiv [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-number-theory WIP 283/0 Mathlib/NumberTheory/Padics/Amice.lean 1 2 ['grunweg'] nobody
63-21594
2 months ago
63-21594
2 months ago
0-0
0 seconds
20671 thefundamentaltheor3m
author:thefundamentaltheor3m
feat(Analysis/Asymptotics/SpecificAsymptotics): Proving that 𝛔ₖ(n) = O(nᵏ⁺¹) This PR proves a result about the $\sigma_k(n)$ arithmetic function, namely, that it is $O\left(n^{k+1}\right)$. Main theorem: `theorem sigma_asymptotic (k : ℕ) : (fun n ↦ (σ k n : ℝ)) =O[atTop] (fun n ↦ (n ^ (k + 1) : ℝ))` This result was proved as part of the sphere packing project. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import new-contributor t-number-theory awaiting-author 29/0 Mathlib/Analysis/Asymptotics/SpecificAsymptotics.lean 1 2 ['b-mehta', 'github-actions'] b-mehta
assignee:b-mehta
63-21305
2 months ago
73-15782
2 months ago
9-59130
9 days
23504 Timeroot
author:Timeroot
feat(ModelTheory/Syntax): substFunc Defines `FirstOrder.Language.Term.substFunc`, a way to substitute function definitions inside of a term. Compare this with existing `subst`, which just substitutes variables. --- Pulled out from #19695 - [ ] depends on: #23502 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-logic blocked-by-other-PR 33/0 Mathlib/ModelTheory/Semantics.lean,Mathlib/ModelTheory/Syntax.lean 2 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
63-18211
2 months ago
63-18213
2 months ago
6-84007
6 days
23790 vasnesterov
author:vasnesterov
feat(Analysis/Analytic): `HasFPowerSeriesOnBall.compContinuousLinearMap` Prove `HasFPowerSeriesOnBall.compContinuousLinearMap` and its variants: if `pf` converges to `f` on the ball `B(u x0, r)` where `u` is continuous linear function, then `pf.compContinuousLinearMap u` converges to `f ∘ u` on `B(x0, r / ‖u‖)`. --- - [ ] depends on: #22531 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis blocked-by-other-PR 216/6 Mathlib/Analysis/Analytic/Basic.lean,Mathlib/Analysis/Analytic/Constructions.lean,Mathlib/Analysis/Calculus/FormalMultilinearSeries.lean,scripts/noshake.json 4 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
63-15570
2 months ago
63-15583
2 months ago
0-1519
25 minutes
19432 mans0954
author:mans0954
feat(LinearAlgebra/QuadraticForm/Basis): Free Tensor product of Quadratic Maps WiP: Define the tensor product of two Quadratic Maps on free modules using `toBilin`. It should then be possible to extend this definition to arbitrary modules using quotients. Similar to `QuadraticMap.tensorDistrib` but without requiring `Invertible (2 : R)`. --- - [x] depends on: #18578 - [x] depends on: #19712 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-algebra WIP
label:t-algebra$
888/0 Mathlib.lean,Mathlib/Data/Sym/Sym2/Prod.lean,Mathlib/LinearAlgebra/QuadraticForm/Basis.lean 3 n/a ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
62-81686
2 months ago
unknown
unknown
21903 yhtq
author:yhtq
feat: add from/toList between `FreeSemigroup` and `List` with relative theorems Add from/toList between `FreeSemigroup` and `List` with relative theorems, as well as an incidental definition of lexicographic order on `FreeSemigroup`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import new-contributor t-algebra awaiting-CI
label:t-algebra$
169/0 Mathlib/Algebra/Free.lean 1 11 ['YaelDillies', 'github-actions'] nobody
62-54115
2 months ago
62-54115
2 months ago
51-9403
51 days
22657 Xmask19
author:Xmask19
feat: a graph is maximally acyclic iff it is a tree --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-combinatorics 86/0 Mathlib/Combinatorics/SimpleGraph/Acyclic.lean 1 6 ['Rida-Hamadani', 'b-mehta', 'github-actions', 'grunweg'] b-mehta
assignee:b-mehta
62-19772
2 months ago
62-19793
2 months ago
84-10469
84 days
23835 chrisflav
author:chrisflav
feat(Topology): cardinality of connected components is bounded by cardinality of fiber --- - [ ] depends on: #23849 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-topology blocked-by-other-PR 302/1 Mathlib.lean,Mathlib/Algebra/BigOperators/Finprod.lean,Mathlib/Data/Set/Card/Arithmetic.lean,Mathlib/Data/Set/Finite/Lattice.lean,Mathlib/Data/Set/Lattice.lean,Mathlib/SetTheory/Cardinal/Finite.lean,Mathlib/Topology/Clopen.lean,Mathlib/Topology/Connected/CardComponents.lean,Mathlib/Topology/Connected/Clopen.lean 9 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
61-74060
2 months ago
61-74062
2 months ago
0-498
8 minutes
23154 vlad902
author:vlad902
feat(Algebra/FreeMonoid): isomorphisms for the free monoid on zero/one generators In parallel to FreeGroup.freeGroupEmptyEquivUnit and FreeGroup.freeGroupUnitEquivInt, prove that the free monoid on zero/one generators is isomorphic to Unit/ℕ. t-algebra awaiting-author
label:t-algebra$
18/0 Mathlib/Algebra/FreeMonoid/Basic.lean 1 2 ['github-actions', 'urkud'] nobody
61-64816
2 months ago
61-64816
2 months ago
19-35867
19 days
23866 kim-em
author:kim-em
chore: remove `[AtLeastTwo n]` hypothesis from the `NatCast` to `OfNat` instance This PR observes that we can change ``` instance (priority := 100) instOfNatAtLeastTwo {n : ℕ} [NatCast R] [Nat.AtLeastTwo n] : OfNat R n ``` to ``` instance (priority := 100) instOfNatAtLeastTwo {n : ℕ} [NatCast R] : OfNat R n ``` with minimal fall-out. A follow-up PR #23867 then observes that we can remove nearly all the `[Nat.AtLeastTwo n]` hypotheses in Mathlib. This is slightly dangerous -- it does make it more likely that we'll generate non-defeq instances, but it appears to happen very rarely. However, it will make life slightly easier for something Leo and I are trying to do with `grind` and Grobner bases (we'd like to be able to assume types we consume have `[∀ n, OfNat α n]`, which is possible with this change, but not without...). Zulip thread: [#PR reviews > #23866 and #23867, removing most `[Nat.AtLeastTwo n]` @ 💬](https://leanprover.zulipchat.com/#narrow/channel/144837-PR-reviews/topic/.2323866.20and.20.2323867.2C.20removing.20most.20.60.5BNat.2EAtLeastTwo.20n.5D.60/near/511157297) awaiting-zulip 21/26 Mathlib/AlgebraicTopology/FundamentalGroupoid/Basic.lean,Mathlib/Data/Nat/Cast/Defs.lean,Mathlib/Data/Nat/Cast/Order/Basic.lean 3 3 ['eric-wieser', 'github-actions', 'urkud'] nobody
61-4028
2 months ago
61-4117
2 months ago
0-23929
6 hours
23186 grunweg
author:grunweg
feat: split continuous linear maps We define split linear maps and prove their basic properties. --- - [ ] depends on #23175 There are two sorries left. One is `ClosedComplemented.prod`; the other relates to the composition of split maps. Help with both is welcome. [This zulip discussion](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Composition.20of.20immersions.20is.20an.20immersion.3A.20infinite-dimensio/with/507300190) contains a proof of the non-trivial sorry. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis WIP help-wanted 240/0 Mathlib.lean,Mathlib/Analysis/NormedSpace/HahnBanach/Splits.lean 2 1 ['github-actions'] nobody
60-13164
1 month ago
60-13164
1 month ago
0-0
0 seconds
21342 YaelDillies
author:YaelDillies
refactor(Normed/Group/Quotient): generalise to non-abelian groups The goal is to apply this to the free group. --- - [x] depends on: #21341 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis WIP 25/12 Mathlib/Topology/Algebra/ConstMulAction.lean,Mathlib/Topology/Algebra/Group/Quotient.lean 2 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
59-45357
1 month ago
59-45376
1 month ago
0-352
5 minutes
19475 YaelDillies
author:YaelDillies
feat: group markings From LeanCamCombi --- - [ ] depends on: #21342 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra blocked-by-other-PR WIP
label:t-algebra$
196/12 Mathlib.lean,Mathlib/Geometry/Group/Marking.lean,Mathlib/Topology/Algebra/ConstMulAction.lean,Mathlib/Topology/Algebra/Group/Quotient.lean 4 12 ['YaelDillies', 'b-mehta', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
59-45291
1 month ago
59-45310
1 month ago
22-16818
22 days
23949 Louddy
author:Louddy
feat: SkewPolynomial # Univariate skew polynomials Skew polynomials are represented as `SkewMonoidAlgebra R (Multiplicative ℕ)`, where `R` is usually at least a Semiring. In this file, we define `SkewPolynomial` and provide basic instances. This is currently missing the definition of `coeff` and `single` as they require a more advance interface of `SkewMonoidAlgebra` which is still WIP (See TODOs in file). Co-authored-by: María Inés de Frutos Fernández <[mariaines.dff@gmail.com](mailto:mariaines.dff@gmail.com)> --- - [ ] depends on: #22078 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import new-contributor t-algebra blocked-by-other-PR
label:t-algebra$
600/42 Mathlib.lean,Mathlib/Algebra/SkewMonoidAlgebra/Basic.lean,Mathlib/Algebra/SkewPolynomial/Basic.lean,docs/references.bib 4 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
59-20722
1 month ago
59-20723
1 month ago
0-2389
39 minutes
18706 FR-vdash-bot
author:FR-vdash-bot
perf: change the priority of `*.toSemiring` instances Need to fix some regressions in subsequent PRs. --- - [ ] depends on: #18468 - [ ] depends on: #18470 From #7873. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-bench slow-typeclass-synthesis t-algebra blocked-by-other-PR WIP
label:t-algebra$
24/15 Mathlib/Algebra/Field/Defs.lean,Mathlib/Algebra/Order/Kleene.lean,Mathlib/Algebra/Ring/Defs.lean,Mathlib/FieldTheory/Extension.lean,Mathlib/FieldTheory/PurelyInseparable.lean,Mathlib/LinearAlgebra/Matrix/Charpoly/Coeff.lean,Mathlib/RingTheory/Etale/Field.lean,Mathlib/RingTheory/Filtration.lean,Mathlib/RingTheory/Localization/Integral.lean 9 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
59-998
1 month ago
214-63136
7 months ago
0-576
9 minutes
18641 FR-vdash-bot
author:FR-vdash-bot
perf: change the priority of `*.toRing` instances --- - [ ] depends on: #18468 - [ ] depends on: #18470 From #7873. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-bench slow-typeclass-synthesis t-algebra blocked-by-other-PR
label:t-algebra$
7/1 Mathlib/Algebra/Field/Defs.lean,Mathlib/Algebra/Ring/BooleanRing.lean,Mathlib/Algebra/Ring/Defs.lean,Mathlib/RingTheory/Valuation/ValuationSubring.lean 4 5 ['FR-vdash-bot', 'github-actions', 'leanprover-bot', 'mathlib4-dependent-issues-bot'] nobody
59-996
1 month ago
216-54247
7 months ago
0-627
10 minutes
20843 mans0954
author:mans0954
feature(Analysis/LocallyConvex/Polar): Bipolar theorem WiP: The Bipolar Theorem Following Conway, Chapter V. 1.8. --- - [x] depends on: #21002 - [ ] depends on: #23845 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis WIP 107/24 Mathlib.lean,Mathlib/Analysis/LocallyConvex/Bipolar.lean,Mathlib/Analysis/Normed/Module/Dual.lean 3 4 ['github-actions', 'j-loreaux', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
58-47863
1 month ago
58-47879
1 month ago
0-0
0 seconds
15420 eric-wieser
author:eric-wieser
feat: port Mathlib 3's `Nat.factors` norm_num extension to a `simproc` This is a partial attempt at #15410, porting [#8009](https://github.com/leanprover-community/mathlib3/pull/8009) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-CI t-meta 190/65 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/NormNum/Prime.lean,Mathlib/Tactic/Simproc/Factors.lean,MathlibTest/factors.lean,MathlibTest/norm_num_ext.lean 6 26 ['Ruben-VandeVelde', 'YaelDillies', 'eric-wieser', 'github-actions', 'kim-em'] nobody
57-70572
1 month ago
57-70614
1 month ago
176-12996
176 days
24010 grunweg
author:grunweg
feat(Counterexamples): a non-negative function, not a.e. zero, with vanishing lowe… …r Lebesgue integral. Came up in #23707, let's document this while we're at it. --- - [ ] depends on: #20722 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-measure-probability please-adopt blocked-by-other-PR WIP 110/0 Counterexamples.lean,Counterexamples/LIntegralZero.lean 2 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
56-85506
1 month ago
56-85508
1 month ago
0-22
22 seconds
24000 YaelDillies
author:YaelDillies
feat: correspondence between Hopf algebras and affine group schemes Construct `Spec` as a functor from `R`-Hopf algebras to group schemes over `Spec R`, show it is full and faithful and has affine group schemes as essential image. From Toric, FLT Co-authored-by: Andrew Yang Co-authored-by: Michał Mrugała Co-authored-by: Christian Merten --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) toric FLT t-algebraic-geometry WIP 127/0 Mathlib/AlgebraicGeometry/GroupScheme/HopfAffine.lean 1 3 ['YaelDillies', 'github-actions', 'kbuzzard'] nobody
56-76754
1 month ago
57-28306
1 month ago
0-1
1 second
21270 GabinKolly
author:GabinKolly
feat(ModelTheory/Bundled): first-order embeddings and equivalences from equalities Add first-order embeddings and equivalences from equalities between bundled structures. --- Add two definitions to get embeddings and equivalences from equalities between bundled structures, and simple properties. This is some preparatory work for #18876 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-logic awaiting-author 102/0 Mathlib/ModelTheory/Bundled.lean 1 26 ['GabinKolly', 'Vierkantor', 'YaelDillies', 'github-actions'] nobody
56-46727
1 month ago
56-46727
1 month ago
50-58472
50 days
21031 YaelDillies
author:YaelDillies
chore: get rid of generic hom coercions --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP 161/168 Mathlib/Algebra/Group/Equiv/Basic.lean,Mathlib/Algebra/Group/Equiv/Defs.lean,Mathlib/Algebra/Group/Hom/Defs.lean,Mathlib/Algebra/Group/Subgroup/Map.lean,Mathlib/Algebra/Group/Units/Hom.lean,Mathlib/Algebra/GroupWithZero/Hom.lean,Mathlib/Algebra/Order/Hom/Monoid.lean,Mathlib/Algebra/Ring/Hom/Defs.lean,Mathlib/GroupTheory/MonoidLocalization/Basic.lean,Mathlib/Logic/Equiv/Defs.lean,Mathlib/Order/Hom/Basic.lean,Mathlib/Order/RelIso/Basic.lean,Mathlib/RingTheory/Valuation/Basic.lean 13 11 ['Vierkantor', 'YaelDillies', 'github-actions', 'leanprover-community-bot-assistant', 'urkud'] nobody
56-38156
1 month ago
59-45489
1 month ago
0-17
17 seconds
20263 joelriou
author:joelriou
feat(CategoryTheory): locally presentable and accessible categories --- - [x] depends on: #19937 - [x] depends on: #19945 - [x] depends on: #19959 - [x] depends on: #20005 - [x] depends on: #19955 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory WIP 220/3 Mathlib.lean,Mathlib/CategoryTheory/Presentable/Basic.lean,Mathlib/CategoryTheory/Presentable/CardinalFilteredPresentation.lean,Mathlib/CategoryTheory/Presentable/LocallyPresentable.lean,Mathlib/SetTheory/Cardinal/HasCardinalLT.lean 5 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
55-47206
1 month ago
55-47304
1 month ago
0-70
1 minute
22367 joelriou
author:joelriou
feat(CategoryTheory/Abelian): Noetherian objects form a Serre class In this PR, we define a type class `IsNoetherianObject X` for any object `X` in a category `C`: it is defined as the ascending chain condition for subobjects of `X`. When `C` is an abelian category, we show that this defines a Serre class. --- This is a draft. - [x] depends on: #22373 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory WIP 311/14 Mathlib.lean,Mathlib/CategoryTheory/Abelian/SerreClass/NoetherianObject.lean,Mathlib/CategoryTheory/Abelian/Subobject.lean,Mathlib/CategoryTheory/Subobject/Basic.lean,Mathlib/CategoryTheory/Subobject/MonoOver.lean 5 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
55-46051
1 month ago
55-46067
1 month ago
0-0
0 seconds
23763 grunweg
author:grunweg
feat(Linter.openClassical): also lint for Classical declarations as … …a local or scoped instance. --- - [ ] depends on: #23750 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-linter 138/33 Mathlib/RingTheory/Perfection.lean,Mathlib/Tactic/Linter/Style.lean,Mathlib/Topology/MetricSpace/GromovHausdorffRealized.lean,MathlibTest/GeneralizeProofs.lean,MathlibTest/LintStyle.lean 5 5 ['github-actions', 'grunweg', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
55-37897
1 month ago
56-30759
1 month ago
56-64979
56 days
24086 mattrobball
author:mattrobball
perf(Normed.Field.Basic): change parent order for `Semifield` and `Field` and reduce priority `toComm(Semi)Ring` Passing through the projection `toComm(Semi)Ring` should not be preferred. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
8/2 Mathlib/Algebra/Field/Defs.lean 1 4 ['github-actions', 'leanprover-bot', 'mattrobball'] nobody
55-13364
1 month ago
55-18164
1 month ago
0-0
0 seconds
13038 adomani
author:adomani
feat: Mathlib weekly reports This PR introduces a weekly cron job that computes a "global" report on the evolution of Mathlib in the previous week. It consists of * a CI workflow with a cron job that runs at minight on Sunday (`.github/workflows/mathlib_stats.yaml`); * a Lean file extracting a categorized list of "all" the declarations in Mathlib (`scripts/count_decls.lean`); * a bash file computing Git-diff-related information and collating the data from the Lean file (`scripts/mathlib_stats.sh`); * a convenience CI workflow that is triggered on adding the `test-ci` label and results in posting on the PR and on Zulip the report (`.github/workflows/mathlib_stats_label.yaml`). The second CI workflow is intended to be removed just before/right after the PR is ready to merge. [Zulip discussion](https://leanprover.zulipchat.com/#narrow/stream/113488-general) [Thread for the reports](https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/Mathlib.20weekly.20change.20report) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) CI t-meta awaiting-author 338/0 .github/workflows/mathlib_stats.yaml,.github/workflows/mathlib_stats_label.yaml,scripts/count_decls.lean,scripts/mathlib_stats.sh 4 10 ['adomani', 'github-actions', 'grunweg', 'kim-em', 'kmill'] nobody
54-80718
1 month ago
329-12198
10 months ago
57-4216
57 days
24112 Vierkantor
author:Vierkantor
fix(Algebra): `MulMemClass.mul_mem` should not be `aesop safe` The `@[aesop safe apply]` attribute only applies to implications that preserve provability. So for `mul_mem (ha : a ∈ s) (hb : b ∈ s) : a * b ∈ s`, there are ways to prove `a * b ∈ s` while `b ∉ s`, such as when `s` is an ideal and `a ∈ s`. So, instead give `MulMemClass.mul_mem` and `AddMemClass.add_mem` the unsafe attribute, and add `Ideal.mul_mem_left` and `Ideal.mul_mem_right` to the aesop with the same `unsafe` attribute. Now we can prove membership of ideals a bit more easily. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
5/1 Mathlib/Algebra/Group/Subsemigroup/Defs.lean,Mathlib/RingTheory/Ideal/Defs.lean 2 1 ['github-actions'] nobody
54-32033
1 month ago
54-32097
1 month ago
54-32080
54 days
24016 plp127
author:plp127
feat: fine uniformity Adds the fine uniformity, and proves some properties. --- - [ ] depends on: #24096 for showing the induced topology is equal on completely regular spaces [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology blocked-by-other-PR 283/0 Mathlib.lean,Mathlib/Topology/UniformSpace/FineUniformity.lean,Mathlib/Topology/UniformSpace/Uniformizable.lean 3 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
53-71737
1 month ago
53-71739
1 month ago
2-85349
2 days
24129 urkud
author:urkud
feat: symmetry of Gateaux derivatives --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis 190/1 Mathlib.lean,Mathlib/Analysis/Calculus/LineDeriv/Basic.lean,Mathlib/Analysis/Calculus/LineDeriv/Symmetric.lean 3 1 ['github-actions'] nobody
53-47945
1 month ago
53-47945
1 month ago
0-0
0 seconds
23637 kirilvino
author:kirilvino
feat(Combinatorics/SimpleGraph): every circuit contains a cycle proof circuit to cycle proof --- This PR uses the bypass definition in a new function for closed walks that removes repeated vertices. Then proves if the closed walk given is a circuit, that the result from this function is a cycle. This is then packaged up similar to the existing ToPath definition, creating a way of transforming a circuit into a cycle. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-combinatorics awaiting-author 26/0 Mathlib/Combinatorics/SimpleGraph/Path.lean 1 8 ['b-mehta', 'github-actions', 'kirilvino'] nobody
53-37204
1 month ago
53-83825
1 month ago
13-19789
13 days
19613 madvorak
author:madvorak
refactor(Combinatorics/Optimization/ValuedCSP): make only valid `FractionalOperation` possible Originally `FractionalOperation` was any multiset (possible empty). Then `FractionalOperation.IsValid` said it was nonempty. Instead, I would like to make it nonempty by definition. As a result, empty/invalid fractional operation couldn't be declared at all. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics 14/17 Mathlib/Combinatorics/Optimization/ValuedCSP.lean 1 1 ['github-actions'] nobody
52-84162
1 month ago
182-19335
6 months ago
192-6980
192 days
22925 ggranberry
author:ggranberry
feat(Mathlib/PlaceHolder/ToeplitzHausdorff): Toeplitz-Hausdorff --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-analysis awaiting-author WIP help-wanted 411/0 Mathlib/PlaceHolder/ToeplitzHausdorff.lean,Mathlib/PlaceHolder/ToeplitzHausdorff_v2.lean 2 10 ['faenuccio', 'ggranberry', 'github-actions'] faenuccio
assignee:faenuccio
52-84002
1 month ago
52-84002
1 month ago
4-24257
4 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/) will-close-soon t-algebra
label:t-algebra$
17/0 Mathlib/FieldTheory/RatFunc/Basic.lean 1 1 ['joneugster'] nobody
52-80776
1 month ago
52-80776
1 month ago
0-0
0 seconds
23600 mattrobball
author:mattrobball
perf(Quiver.Basic): make `IsThin` a `class` It seems problematic that `Quiver.IsThin` is an `abbrev` for (essentially) `Subsingleton`. We turn it in a one-field class. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) delegated 27/21 Mathlib/CategoryTheory/Bicategory/Coherence.lean,Mathlib/CategoryTheory/Category/Preorder.lean,Mathlib/CategoryTheory/Generator/Basic.lean,Mathlib/CategoryTheory/Groupoid/Basic.lean,Mathlib/CategoryTheory/Limits/Shapes/WidePullbacks.lean,Mathlib/CategoryTheory/Limits/SmallComplete.lean,Mathlib/CategoryTheory/Monoidal/Free/Coherence.lean,Mathlib/CategoryTheory/Skeletal.lean,Mathlib/CategoryTheory/Subobject/MonoOver.lean,Mathlib/CategoryTheory/Thin.lean,Mathlib/Combinatorics/Quiver/Basic.lean 11 16 ['b-mehta', 'github-actions', 'leanprover-bot', 'mathlib-bors', 'mattrobball'] nobody
52-14897
1 month ago
67-13701
2 months ago
0-5717
1 hour
12561 BoltonBailey
author:BoltonBailey
doc: suggest !bench in `lake exe pole` This change explains what to do if the benchmarks haven't been run. --- - [x] depends on: #12322 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 2/1 LongestPole/Main.lean 1 2 ['github-actions', 'leanprover-community-mathlib4-bot'] nobody
50-67996
1 month ago
unknown
unknown
24218 alreadydone
author:alreadydone
chore(Algebra): remove `mid_assoc` from `IsMulCentral` as it is a consequence of left and right associativity in the presence of commutativity. Also change the commutativity condition to use `Commute`. --- Even without commutativity, left and right associativity of an element `e` in a magma is sufficient to prove that elements of the form `e * x * e` (the "corner" of `e`) form a submagma. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
31/69 Mathlib/Algebra/Algebra/NonUnitalSubalgebra.lean,Mathlib/Algebra/Group/Center.lean,Mathlib/Algebra/GroupWithZero/Center.lean,Mathlib/Algebra/Ring/Center.lean,Mathlib/Algebra/Ring/CentroidHom.lean,Mathlib/Algebra/Star/Center.lean,Mathlib/Algebra/Star/CentroidHom.lean,Mathlib/GroupTheory/Submonoid/Center.lean,Mathlib/LinearAlgebra/Basis/Submodule.lean,Mathlib/LinearAlgebra/QuadraticForm/Basic.lean,Mathlib/RingTheory/Idempotents.lean,Mathlib/RingTheory/NonUnitalSubsemiring/Basic.lean 12 8 ['alreadydone', 'github-actions', 'mans0954'] nobody
50-12169
1 month ago
50-27229
1 month ago
50-27219
50 days
23990 robertmaxton42
author:robertmaxton42
feat (Types.Colimits): Quot is functorial and colimitEquivQuot is natural Add `Functor.quotFunctor` to parallel `Functor.sectionsFunctor`, witnessing that `Quot` is functorial; add `colimNatIsoQuotFunctor` to parallel `limNatIsoSectionsFunctor`, witnessing that `colimitEquivQuot` is natural in the diagram $F$. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-category-theory awaiting-author 33/0 Mathlib/CategoryTheory/Limits/Types/Colimits.lean 1 4 ['github-actions', 'joelriou', 'robertmaxton42'] nobody
49-15397
1 month ago
49-15397
1 month ago
8-28043
8 days
20689 joelriou
author:joelriou
feat(AlgebraicTopology): cylinder objects in model categories --- - [x] depends on: #20666 - [x] depends on: #20680 - [ ] depends on: #20210 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-category-theory blocked-by-other-PR WIP 820/4 Mathlib.lean,Mathlib/AlgebraicTopology/ModelCategory/Basic.lean,Mathlib/AlgebraicTopology/ModelCategory/Cylinder.lean,Mathlib/AlgebraicTopology/ModelCategory/Instances.lean,Mathlib/AlgebraicTopology/ModelCategory/IsFibrant.lean 5 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
49-6791
1 month ago
49-6810
1 month ago
0-0
0 seconds
24219 Paul-Lez
author:Paul-Lez
feat: linear independence of the tensor product of two linearly independent families This is still WIP (the proofs are a little too long, and some lemmas need to be moved to other files!) From Toric --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) toric t-algebra WIP
label:t-algebra$
193/0 Mathlib/LinearAlgebra/LinearIndependent/Tprod.lean 1 1 ['github-actions'] nobody
48-16595
1 month ago
48-16595
1 month ago
0-2221
37 minutes
22898 AntoineChambert-Loir
author:AntoineChambert-Loir
feat(RingTheory/TensorProduct/DirectLimit/FG): direct limit of finitely generated submodules and tensor product --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra WIP
label:t-algebra$
399/0 Mathlib.lean,Mathlib/RingTheory/Adjoin/FG.lean,Mathlib/RingTheory/Finiteness/Basic.lean,Mathlib/RingTheory/TensorProduct/Basic.lean,Mathlib/RingTheory/TensorProduct/DirectLimit/FG.lean 5 8 ['AntoineChambert-Loir', 'alreadydone', 'github-actions'] nobody
47-80925
1 month ago
77-18612
2 months ago
11-9349
11 days
21582 jjdishere
author:jjdishere
feat(RingTheory/AdicCompletion): more APIs for IsAdicComplete In this PR, we establish more APIs for IsAdicComplete. 1. Instead of checking the definition in `IsPrecomplete` (starting with a compatible sequence in M), we build APIs to lift elements (or maps) from compatible sequences in `M ⧸ I ^ n • ⊤`. 2. We also build APIs to lift a sequence of `LinearMap`s to `LinearMap` and a sequence of `RingHom`s to `RingHom` directly. 3. Since `I * ⊤` is not definitionally equal to `I`, we build special APIs for the `M = R` case, enabling one to use `R ⧸ I ^ n` instead of `R ⧸ I ^ n • ⊤`. 4. We generalize the compatible sequence from defined on every `M ⧸ I ^ n • ⊤` to only defined on `M ⧸ I ^ a n • ⊤` for a strictly increasing sequence `a n`. (I would use the case `a n = n + 1` in #21564 ) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra awaiting-author
label:t-algebra$
388/10 Mathlib/RingTheory/AdicCompletion/Basic.lean,Mathlib/RingTheory/Ideal/Quotient/Defs.lean,Mathlib/RingTheory/Ideal/Quotient/PowTransition.lean 3 17 ['github-actions', 'jjdishere', 'mergify', 'riccardobrasca'] riccardobrasca
assignee:riccardobrasca
47-46078
1 month ago
47-46094
1 month ago
13-38587
13 days
13740 YaelDillies
author:YaelDillies
feat: More robust ae notation Make sure that, when `μ : FiniteMeasure Ω`, `f =ᵐ[μ] g` elaborates to `f =ᵐ[↑μ] g` instead of complaining about `OuterMeasureClass (FiniteMeasure Ω) (Set Ω) ℝ≥0∞` not existing. [Zulip](https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/ae.20of.20a.20finite.20measure) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-measure-probability awaiting-CI t-meta 56/2 Mathlib/MeasureTheory/Measure/MeasureSpaceDef.lean,Mathlib/MeasureTheory/OuterMeasure/AE.lean,Mathlib/MeasureTheory/OuterMeasure/BorelCantelli.lean 3 16 ['YaelDillies', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'urkud'] nobody
47-41067
1 month ago
47-41082
1 month ago
0-0
0 seconds
24161 urkud
author:urkud
feat(Analysis/Calculus/Schwarzian): new file --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis 190/3 Mathlib.lean,Mathlib/Analysis/Calculus/Deriv/ZPow.lean,Mathlib/Analysis/Calculus/Schwarzian/Basic.lean 3 2 ['github-actions', 'leanprover-community-bot-assistant'] nobody
47-27921
1 month ago
47-27939
1 month ago
0-0
0 seconds
20409 vihdzp
author:vihdzp
feat: linear order is isomorphic to lexicographic sum of two intervals --- The material in this PR was previously in #18893. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order awaiting-CI 169/2 Mathlib.lean,Mathlib/Data/Sum/Order.lean,Mathlib/Logic/Equiv/Set.lean,Mathlib/Order/Hom/Lex.lean,Mathlib/Order/Hom/Set.lean 5 21 ['YaelDillies', 'eric-wieser', 'github-actions', 'vihdzp'] nobody
47-20770
1 month ago
47-20770
1 month ago
109-5714
109 days
20652 jjaassoonn
author:jjaassoonn
feat: categorical description of center of a ring We show the isomorphism between `Z(R)` and `End(1 Mod-R)` --- - [x] depends on:#20721 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-category-theory awaiting-author
label:t-algebra$
212/21 Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/ChangeOfRings.lean,Mathlib/Algebra/Category/Ring/Center.lean,Mathlib/CategoryTheory/Conj.lean,Mathlib/CategoryTheory/Endomorphism.lean,Mathlib/CategoryTheory/Preadditive/AdditiveFunctor.lean,Mathlib/CategoryTheory/Preadditive/Basic.lean 7 41 ['alreadydone', 'github-actions', 'jcommelin', 'jjaassoonn', 'kbuzzard', 'qawbecrdtey'] nobody
46-70433
1 month ago
104-36114
3 months ago
20-7596
20 days
10655 BoltonBailey
author:BoltonBailey
feat: one time pad string diagram String-diagrammatic proof of OTP --- - [x] depends on: #10581 [Defines the diagram widget] [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 159/0 MathlibTest/StringDiagram.lean 1 2 ['github-actions', 'leanprover-community-mathlib4-bot'] nobody
46-63653
1 month ago
unknown
unknown
21616 peabrainiac
author:peabrainiac
feat(Topology): concatenating countably many paths Adds `Path.countableConcat`, the concatenation of a sequence of paths leading up to some point `x`. --- - [x] depends on: #21591 - [x] depends on: #21607 This work is a prerequisite to #20248, where it is used to show that the topology of first-countable locally path-connected spaces is coinduced by all the paths in that space. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology awaiting-author 229/0 Mathlib.lean,Mathlib/Topology/Path/CountableConcat.lean 2 30 ['YaelDillies', 'github-actions', 'kim-em', 'mathlib4-dependent-issues-bot', 'peabrainiac'] YaelDillies
assignee:YaelDillies
46-36356
1 month ago
50-44290
1 month ago
56-56728
56 days
18210 vihdzp
author:vihdzp
feat(Order/Hom/Basic): `WithBot (Fin n) ≃o Fin (n + 1)` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order awaiting-author 16/0 Mathlib/Order/Hom/Basic.lean 1 8 ['Command-Master', 'Ruben-VandeVelde', 'github-actions', 'urkud', 'vihdzp'] nobody
45-69064
1 month ago
216-73142
7 months ago
10-77913
10 days
23585 plp127
author:plp127
feat: `Filter.atMax` and `Filter.atMin` Adds `atMax` and `atMin`, filters. Making an analogy, `atMax` : `atTop` :: `IsMax` : `IsTop`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order WIP 148/0 Mathlib.lean,Mathlib/Order/Filter/AtMaxMin.lean 2 4 ['github-actions', 'plp127', 'urkud'] nobody
45-59873
1 month ago
68-34531
2 months ago
0-0
0 seconds
23026 Paul-Lez
author:Paul-Lez
feat(Tactic/Simproc/Divisors): add `simproc`s to compute the divisors of a natural number. We add some `simproc`s to compute the `Nat.divisors` and `Nat.properDivisors`. Co-authored-by: Bhavik Mehta --- - [x] depends on: #23025 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta awaiting-author 83/0 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Simproc/Divisors.lean,MathlibTest/Simproc/Divisors.lean 4 26 ['Paul-Lez', 'b-mehta', 'eric-wieser', 'github-actions', 'j-loreaux', 'mathlib4-dependent-issues-bot'] nobody
44-58201
1 month ago
44-58201
1 month ago
9-45842
9 days
22349 dtumad
author:dtumad
feat(Control): Laws for monads with compatible `failure` operation Add a class for a `Monad` that also has an `Alternative` instance, and a class `LawfulAlternative` for types where the failure and monad structures are compatible in the expected way. --- I'm not sure if this should instead go in `Batteries.Control` instead of mathlib, or at least lemmas like `OptionT.run_failure` maybe should. Some of the instances like `Set` would still need to be added in mathlib either way. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-meta WIP 74/3 Mathlib.lean,Mathlib/Control/Lawful.lean,Mathlib/Control/Monad/AlternativeMonad.lean 3 8 ['dtumad', 'eric-wieser', 'github-actions', 'quangvdao'] nobody
44-55296
1 month ago
44-55450
1 month ago
1-20563
1 day
24394 wwylele
author:wwylele
feat(Analysis/Asymptotics): Add filter operation theorems to `IsEquivalent` These are simply restating the corresponding theorems for `isLittleO`, but adding them provides better discovery when one is not familiar with how `IsEquivalent` is defined. I tagged `isEquivalent_map` as `@[simp]` because all of `isBigOWith/isBigO/isLittleO_map` are tagged, but I am not sure if this appropriate. Please let me know if I should remove the tag --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-analysis 13/0 Mathlib/Analysis/Asymptotics/AsymptoticEquivalent.lean 1 1 ['github-actions'] nobody
44-3314
1 month ago
44-3314
1 month ago
44-3373
44 days
22547 joelriou
author:joelriou
feat(CategoryTheory/Abelian): construction of reduced left resolutions The standard functorial free resolution of a `R`-module `M` does not directly extend to free resolutions of (bounded above) complexes because the free `R`-module functor does preserve zero morphisms. In this PR, we provide a general construction which takes functorial left resolutions and modify them by considering a suitable direct factor so that it preserves zero morphisms. --- - [ ] depends on: #22539 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory blocked-by-other-PR WIP 514/19 Mathlib.lean,Mathlib/Algebra/Homology/HomologicalComplex.lean,Mathlib/Algebra/Homology/LeftResolutions/Basic.lean,Mathlib/Algebra/Homology/LeftResolutions/Reduced.lean,Mathlib/Algebra/Homology/LeftResolutions/Transport.lean,Mathlib/CategoryTheory/Limits/Shapes/Kernels.lean 6 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
43-2573
1 month ago
97-24888
3 months ago
0-358
5 minutes
22556 joelriou
author:joelriou
feat(Algebra/Category/ModuleCat): a functorial projective resolution --- - [ ] depends on: #22539 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory blocked-by-other-PR 315/19 Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/LeftResolutions.lean,Mathlib/Algebra/Homology/HomologicalComplex.lean,Mathlib/Algebra/Homology/LeftResolutions/Basic.lean,Mathlib/CategoryTheory/Limits/Shapes/Kernels.lean 5 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
43-2443
1 month ago
97-19201
3 months ago
0-516
8 minutes
12032 mcdoll
author:mcdoll
feat: Delta distribution as a limit --- - [x] depends on: #11496 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis WIP 51/0 Mathlib/Analysis/Distribution/DiracDelta.lean 1 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
42-74668
1 month ago
unknown
unknown
24405 mcdoll
author:mcdoll
refactor(Topology/Algebra/Module/WeakDual): Clean up - Move `Dual` and `dualPairing` lower in the import-hierachy - deduplicate `dualPairing` - Make `WeakDual` and `WeakSpace` reducible --- New version of #11500 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-topology 146/162 Mathlib.lean,Mathlib/Analysis/Fourier/RiemannLebesgueLemma.lean,Mathlib/Analysis/InnerProductSpace/Adjoint.lean,Mathlib/Analysis/InnerProductSpace/Dual.lean,Mathlib/Analysis/LocallyConvex/WeakSpace.lean,Mathlib/Analysis/Normed/Module/Dual.lean,Mathlib/Analysis/Normed/Module/WeakDual.lean,Mathlib/Analysis/VonNeumannAlgebra/Basic.lean,Mathlib/MeasureTheory/Function/AEEqOfIntegral.lean,Mathlib/MeasureTheory/Measure/FiniteMeasure.lean,Mathlib/Topology/Algebra/Module/Dual.lean,Mathlib/Topology/Algebra/Module/WeakDual.lean,docs/overview.yaml,docs/undergrad.yaml 14 1 ['github-actions'] nobody
42-65841
1 month ago
42-74534
1 month ago
42-74517
42 days
23528 Ruben-VandeVelde
author:Ruben-VandeVelde
feat: add isOpen_setOf_affineIndependent From sphere-eversion. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis delegated 15/0 Mathlib/Analysis/Normed/Module/FiniteDimension.lean 1 3 ['github-actions', 'mathlib-bors', 'urkud'] nobody
42-55626
1 month ago
42-55627
1 month ago
26-70139
26 days
24445 kbuzzard
author:kbuzzard
chore: remove outParam from Valued --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) Exploring the idea that Gamma_0 should not be an outParam in Valued. t-topology WIP 4/3 Mathlib/Topology/Algebra/Valued/ValuationTopology.lean 1 2 ['erdOne', 'github-actions'] nobody
41-39786
1 month ago
41-42270
1 month ago
0-0
0 seconds
9915 eric-wieser
author:eric-wieser
refactor: Add norm_num machinery for NNRat This splits the previous `isRat` primitive into `isNNRat` and `isNegNNRat`, where only the latter carries around a `DivisionRing` instance. This means that `norm_num` works on `NNReal` and `NNRat`. --- - [x] depends on: #9951 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-meta please-adopt WIP
label:t-algebra$
732/211 Mathlib/Analysis/SpecialFunctions/Log/Basic.lean,Mathlib/Analysis/SpecialFunctions/Pow/Real.lean,Mathlib/Data/Rat/Floor.lean,Mathlib/Tactic/NormNum/Basic.lean,Mathlib/Tactic/NormNum/BigOperators.lean,Mathlib/Tactic/NormNum/Eq.lean,Mathlib/Tactic/NormNum/Ineq.lean,Mathlib/Tactic/NormNum/Inv.lean,Mathlib/Tactic/NormNum/OfScientific.lean,Mathlib/Tactic/NormNum/Pow.lean,Mathlib/Tactic/NormNum/RealSqrt.lean,Mathlib/Tactic/NormNum/Result.lean,Mathlib/Tactic/Positivity/Core.lean,Mathlib/Tactic/Ring/Basic.lean,Mathlib/Tactic/Ring/RingNF.lean,MathlibTest/norm_num.lean,MathlibTest/ring.lean 17 3 ['github-actions', 'leanprover-community-mathlib4-bot', 'plp127'] nobody
41-29360
1 month ago
43-74088
1 month ago
0-0
0 seconds
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/) large-import t-algebra blocked-by-other-PR
label:t-algebra$
356/2 Mathlib.lean,Mathlib/Data/Nat/Factorial/NatCast.lean,Mathlib/RingTheory/DividedPowers/RatAlgebra.lean 3 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
41-26426
1 month ago
41-26428
1 month ago
2-68902
2 days
24157 urkud
author:urkud
feat(Convex/LinearIsometry): new file --- - [x] depends on: #24392 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis awaiting-author 75/0 Mathlib.lean,Mathlib/Analysis/Convex/LinearIsometry.lean 2 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'sgouezel'] nobody
40-41601
1 month ago
40-41601
1 month ago
10-23076
10 days
20210 joelriou
author:joelriou
feat(AlgebraicTopology): application of the retract argument to model categories Basic consequences of the retract argument are obtained for model categories: cofibrations are exactly the morphisms that have the left lifting property with respect to trivial fibrations, etc. We deduce various properties of cofibrations, fibrations and weak equivalences in model categories (e.g. they are stable by composition). --- - [x] depends on: #19158 - [x] depends on: #20666 - [x] depends on: #20680 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-category-theory WIP 440/4 Mathlib.lean,Mathlib/AlgebraicTopology/ModelCategory/Basic.lean,Mathlib/AlgebraicTopology/ModelCategory/Instances.lean 3 3 ['github-actions', 'joelriou', 'mathlib4-dependent-issues-bot'] nobody
40-31248
1 month ago
64-36101
2 months ago
0-46563
12 hours
24411 joelriou
author:joelriou
feat(CategoryTheory): descent of morphisms for a pseudofunctor Let `C` be a category and `F : Pseudofunctor (LocallyDiscrete Cᵒᵖ) Cat`. Given `S : C`, and objects `M` and `N` in `F.obj (.mk (op S))`, we define a presheaf of types `F.presheafHom M N` on the category `Over S`: its sections on a object `T : Over S` corresponding to a morphism `p : X ⟶ S` are the type of morphisms `p^* M ⟶ p^* N`. We shall say that `F` satisfies the descent of morphisms for a Grothendieck topology `J` if these presheaves are all sheaves (typeclass `F.HasDescentOfMorphisms J`). Co-authored-by: Christian Merten [christian@merten.dev](mailto:christian@merten.dev) --- - [ ] depends on: #24382 - [ ] depends on: #24384 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory blocked-by-other-PR WIP 474/0 Mathlib.lean,Mathlib/CategoryTheory/Bicategory/Functor/Cat.lean,Mathlib/CategoryTheory/Bicategory/Functor/Strict.lean,Mathlib/CategoryTheory/Sites/Descent/Morphisms.lean 4 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
40-30882
1 month ago
40-30884
1 month ago
0-0
0 seconds
19444 joelriou
author:joelriou
feat(CategoryTheory/Sites): Equivalence of categories of sheaves with a dense subsite that is 1-hypercover dense The main result is that if `F : C₀ ⥤ C` is a dense subsite (relatively to topologies `J₀` and `J`) and `F.IsOneHypercoverDense J₀ J` (for a certain universe `w`), then if a coefficient category `A` has limits of size `w`, the pushforward functor induces an equivalence `Sheaf J A ≌ Sheaf J₀ A`. We deduce that if `HasSheafify J₀ A`, then `HasSheafify J A` also holds. This was previously known (see `IsDenseSubsite.sheafEquiv` in `Sites.DenseSubsite`) under a somewhat stronger condition about the existence of limits in `A`. --- - [x] depends on: #19517 - [x] depends on: #19519 This is very much a draft. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory WIP 937/2 Mathlib.lean,Mathlib/CategoryTheory/Sites/Continuous.lean,Mathlib/CategoryTheory/Sites/DenseSubsite/Basic.lean,Mathlib/CategoryTheory/Sites/DenseSubsite/OneHypercoverDense.lean,Mathlib/CategoryTheory/Sites/DenseSubsite/SheafEquiv.lean,Mathlib/CategoryTheory/Sites/OneHypercover.lean 6 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
40-30116
1 month ago
45-85405
1 month ago
0-0
0 seconds
24489 mattrobball
author:mattrobball
test 185/152 Mathlib/Algebra/GCDMonoid/Nat.lean,Mathlib/Algebra/Group/Defs.lean,Mathlib/Algebra/GroupWithZero/Defs.lean,Mathlib/Algebra/Polynomial/Coeff.lean,Mathlib/Algebra/Polynomial/Eval/Degree.lean,Mathlib/Algebra/Polynomial/Monic.lean,Mathlib/Algebra/Ring/Defs.lean,Mathlib/AlgebraicGeometry/AffineSpace.lean,Mathlib/Analysis/CStarAlgebra/Classes.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Integral.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Isometric.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Unique.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Unital.lean,Mathlib/Analysis/Complex/Polynomial/Basic.lean,Mathlib/Analysis/InnerProductSpace/Adjoint.lean,Mathlib/Analysis/Normed/Algebra/Spectrum.lean,Mathlib/Analysis/NormedSpace/PiTensorProduct/InjectiveSeminorm.lean,Mathlib/Data/Nat/Bitwise.lean,Mathlib/Data/Nat/Choose/Vandermonde.lean,Mathlib/FieldTheory/Galois/Profinite.lean,Mathlib/FieldTheory/IsAlgClosed/Spectrum.lean,Mathlib/FieldTheory/KummerExtension.lean,Mathlib/FieldTheory/KummerPolynomial.lean,Mathlib/GroupTheory/SpecificGroups/Cyclic.lean,Mathlib/GroupTheory/SpecificGroups/Dihedral.lean,Mathlib/GroupTheory/Subgroup/Center.lean,Mathlib/LinearAlgebra/CliffordAlgebra/Basic.lean,Mathlib/LinearAlgebra/CliffordAlgebra/Grading.lean,Mathlib/LinearAlgebra/ExteriorAlgebra/Grading.lean,Mathlib/LinearAlgebra/Matrix/SpecialLinearGroup.lean,Mathlib/LinearAlgebra/PiTensorProduct.lean,Mathlib/LinearAlgebra/RootSystem/Finite/CanonicalBilinear.lean,Mathlib/NumberTheory/NumberField/CanonicalEmbedding/Basic.lean,Mathlib/RepresentationTheory/FDRep.lean,Mathlib/RingTheory/Spectrum/Prime/ChevalleyComplexity.lean,Mathlib/RingTheory/Valuation/ValuationSubring.lean,Mathlib/RingTheory/WittVector/Frobenius.lean,Mathlib/Tactic/Ring/Basic.lean 38 4 ['github-actions', 'leanprover-bot', 'mattrobball'] nobody
39-81726
1 month ago
39-84159
1 month ago
0-0
0 seconds
20719 gio256
author:gio256
feat(AlgebraicTopology): delaborators for truncated simplicial notations We add delaborators for the following notations, introduced in #20688: - `⦋m⦌ₙ`, which denotes the `m`-dimensional simplex in the `n`-truncated simplex category. - `X _⦋m⦌ₙ`, which denotes the `m`-th term of an `n`-truncated simplicial object `X`. - `X ^⦋m⦌ₙ`, which denotes the `m`-th term of an `n`-truncated cosimplicial object `X`. If `pp.proofs` is set to `true`, we also pretty-print the proof `p : m ≤ n` for all three notations as `⦋m, p⦌ₙ`, `X _⦋m, p⦌ₙ`, and `X ^⦋m, p⦌ₙ`, respectively. Credit to @kmill for one piece of code and much metaprogramming inspiration. --- - [x] depends on: #20688 - [x] depends on: #23018 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) infinity-cosmos t-category-theory t-meta 525/33 Mathlib.lean,Mathlib/AlgebraicTopology/SimplexCategory/Basic.lean,Mathlib/AlgebraicTopology/SimplexCategory/Defs.lean,Mathlib/AlgebraicTopology/SimplicialObject/Basic.lean,Mathlib/Tactic.lean,Mathlib/Tactic/SimplexCategory.lean,Mathlib/Util/Superscript.lean,MathlibTest/SimplexCategory.lean,MathlibTest/SimplicialObject.lean,MathlibTest/superscript.lean,scripts/noshake.json 11 22 ['eric-wieser', 'gio256', 'github-actions', 'kim-em', 'mathlib4-dependent-issues-bot'] eric-wieser
assignee:eric-wieser
39-7178
1 month ago
39-9819
1 month ago
47-81361
47 days
14203 dagurtomas
author:dagurtomas
feat(Algebra/ModuleCat): descent data Co-authored-by: Jack McKoen Co-authored-by: Christian Merten Co-authored-by: Joël Riou Co-authored-by: Adam Topaz --- - [ ] depends on: #24530 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) workshop-AIM-AG-2024 t-algebra t-algebraic-geometry t-category-theory blocked-by-other-PR WIP
label:t-algebra$
253/15 Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/ChangeOfRings.lean,Mathlib/Algebra/Category/ModuleCat/Descent.lean,Mathlib/Algebra/Homology/ShortComplex/ExactFunctor.lean,Mathlib/Algebra/Ring/Equiv.lean,Mathlib/AlgebraicGeometry/Morphisms/RingHomProperties.lean,Mathlib/RingTheory/Flat/FaithfullyFlat/Basic.lean,Mathlib/RingTheory/LocalProperties/Basic.lean,Mathlib/RingTheory/RingHom/FaithfullyFlat.lean,Mathlib/RingTheory/RingHom/Finite.lean,Mathlib/RingTheory/RingHom/Flat.lean,Mathlib/RingTheory/RingHom/Integral.lean,Mathlib/RingTheory/RingHom/Locally.lean,Mathlib/RingTheory/RingHom/Surjective.lean,Mathlib/RingTheory/RingHom/Unramified.lean,Mathlib/RingTheory/RingHomProperties.lean 16 3 ['dagurtomas', 'github-actions', 'mathlib4-dependent-issues-bot'] nobody
38-71561
1 month ago
38-71563
1 month ago
0-0
0 seconds
24558 mattrobball
author:mattrobball
test 32/30 Mathlib/Analysis/Analytic/Basic.lean,Mathlib/Analysis/Calculus/ContDiff/Defs.lean,Mathlib/Data/Matroid/Circuit.lean,Mathlib/Data/Matroid/Closure.lean,Mathlib/Data/Matroid/Loop.lean,Mathlib/Data/Set/Insert.lean,Mathlib/FieldTheory/IntermediateField/Adjoin/Basic.lean,Mathlib/Geometry/Euclidean/Angle/Oriented/Affine.lean,Mathlib/Geometry/Euclidean/Angle/Unoriented/Affine.lean,Mathlib/Geometry/Manifold/ContMDiff/Defs.lean,Mathlib/LinearAlgebra/AffineSpace/FiniteDimensional.lean,Mathlib/Order/Cover.lean 12 4 ['github-actions', 'leanprover-bot', 'mattrobball'] nobody
38-12041
1 month ago
38-14901
1 month ago
0-0
0 seconds
24266 plp127
author:plp127
feat(Order): `NoBotOrder α` implies `NoMinOrder α` under `IsDirected α (· ≥ ·)` Proves that `NoBotOrder α` implies `NoMinOrder α` under `IsDirected α (· ≥ ·)`, and also the dual theorem. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order 14/0 Mathlib/Order/Directed.lean 1 4 ['github-actions', 'plp127', 'urkud'] nobody
37-63061
1 month ago
48-74442
1 month ago
48-74426
48 days
18861 YaelDillies
author:YaelDillies
refactor: make `Set.mem_graphOn` defeq The definition as an image is cute but not very useful. Also unsimp `graphOn_univ` since the RHS contains `f` more times than the LHS does. --- Later, I would like to introduce `Set.graph` to have a `Set` version with good defeqs of `LinearMap.graph` and alike [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data awaiting-author 72/18 Mathlib/Data/Set/Function.lean,Mathlib/Data/Set/Operations.lean,Mathlib/Data/Set/Prod.lean,Mathlib/MeasureTheory/Covering/Besicovitch.lean 4 4 ['YaelDillies', 'b-mehta', 'github-actions'] nobody
37-49341
1 month ago
78-2650
2 months ago
2-24624
2 days
23498 Ruben-VandeVelde
author:Ruben-VandeVelde
chore(Topology.MetricSpace.Lipschitz): stop depending on Topology.Algebra Noticed while playing with the new `directoryDependency` linter. Not sure if these could be proved without assuming the continuity of real multiplication. Copyright from https://github.com/leanprover-community/mathlib3/pull/1921 and https://github.com/leanprover-community/mathlib4/pull/11840. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology 60/34 Mathlib.lean,Mathlib/Analysis/Normed/Group/AddTorsor.lean,Mathlib/Analysis/NormedSpace/Multilinear/Basic.lean,Mathlib/Analysis/SpecialFunctions/Exp.lean,Mathlib/Topology/Algebra/MetricSpace/Lipschitz.lean,Mathlib/Topology/MetricSpace/Algebra.lean,Mathlib/Topology/MetricSpace/IsometricSMul.lean,Mathlib/Topology/MetricSpace/Lipschitz.lean,Mathlib/Topology/MetricSpace/PiNat.lean 9 1 ['github-actions'] nobody
37-46198
1 month ago
37-46198
1 month ago
70-25921
70 days
23360 kim-em
author:kim-em
chore: review of `erw` in `Algebra/Homology/DerivedCategory` t-algebra
label:t-algebra$
21/15 Mathlib/Algebra/Homology/DerivedCategory/Basic.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/ExtClass.lean,Mathlib/Algebra/Homology/DerivedCategory/SingleTriangle.lean,Mathlib/Algebra/Homology/HomotopyCategory/SingleFunctors.lean,Mathlib/CategoryTheory/Shift/SingleFunctors.lean 5 2 ['Ruben-VandeVelde', 'github-actions'] nobody
37-46186
1 month ago
37-46186
1 month ago
74-57653
74 days
23503 apnelson1
author:apnelson1
feat(Topology/Instances/ENat): ENat and tsum We give API for the interactions between `tsum` and `ENat`. The type is especially nice, because every function is summable, and there are simplifying lemmas like the statement that a sum is infinite iff either some term is infinite, or the support is infinite. This provides one of the missing pieces for working painlessly with discrete objects, 'propositional' finiteness and cardinality. For instance, one can sum a function `f : a -> ENat` over an arbitrary set with the term `∑' a : s, 1`, and it will be provable that `∑' a : s, 1 = s.encard` and `(support f).encard ≤ ∑' a, f a` without ever having to split into finite/infinite cases. As is pointed out in the module docstring for `Data.ENat`, there are strong analogies between `ENat` and `ENNReal`, and the API runs parallel to the API for `tsum`/`ENNReal`. One could call it 'duplication', but I have yet to find a common generalization of the two that saves work, or a third example of a natural type with these same properties. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-topology WIP 205/2 Mathlib/Data/ENat/Basic.lean,Mathlib/Data/Set/Card.lean,Mathlib/Topology/Instances/ENat.lean 3 2 ['eric-wieser', 'github-actions'] nobody
37-45222
1 month ago
37-45222
1 month ago
14-6036
14 days
22809 b-reinke
author:b-reinke
feat: Category algebras and path algebras This PR defines the category algebra of a linear category and path algebras of quivers. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra t-category-theory WIP
label:t-algebra$
218/0 Mathlib/Algebra/Ring/Assoc.lean,Mathlib/CategoryTheory/Linear/CategoryAlgebra.lean,Mathlib/Combinatorics/Quiver/PathAlgebra.lean,Mathlib/Data/DFinsupp/BigOperators.lean 4 2 ['b-reinke', 'github-actions'] nobody
37-45186
1 month ago
37-45186
1 month ago
0-0
0 seconds
21776 alreadydone
author:alreadydone
Invertible modules --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
571/26 Mathlib/Algebra/Algebra/Operations.lean,Mathlib/Algebra/Module/Submodule/Equiv.lean,Mathlib/Data/Set/Semiring.lean,Mathlib/RingTheory/FractionalIdeal/Operations.lean,Mathlib/RingTheory/PicardGroup.lean 5 2 ['alreadydone', 'github-actions'] nobody
37-45119
1 month ago
37-45119
1 month ago
0-0
0 seconds
19797 eric-wieser
author:eric-wieser
refactor: use Qq in the nlinarith preprocessor This also provides the machinery needed to Qq-ify linarith itself. This is still doing far more `synthInstanceQ`/`isDefEq`(`Q`) than should be needed, but at least drops the `mkAppM`s. Currently, this takes a different approach to the one used by `NormNum.Result`: * `NormNum.Result` deliberately avoids adding any `Expr` parameters to types, as this makes defeq problem at compile-time hard * This PR allows the Expr parameters, but adds casting helpers to easily transport along defeq(Q)s. A few `unsafeIntro`s are left, which correspond to either a Qq bug, or a flaw in the idea behind this approach. I don't know if this pattern is an improvement. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-meta 260/28 Mathlib/Data/Ineq.lean,Mathlib/Tactic/Linarith/Datatypes.lean,Mathlib/Tactic/Linarith/Oracle/SimplexAlgorithm.lean,Mathlib/Tactic/Linarith/Preprocessing.lean,Mathlib/Util/Qq.lean 5 8 ['eric-wieser', 'github-actions', 'leanprover-bot'] nobody
37-44908
1 month ago
37-44908
1 month ago
0-0
0 seconds
14348 eric-wieser
author:eric-wieser
perf: disable the `unusedVariables` linter for speed I doubt we want to merge this, but it shaves two minutes of the lint time. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) performance-hack 1/0 lakefile.lean 1 3 ['eric-wieser', 'github-actions', 'leanprover-bot'] nobody
37-44216
1 month ago
37-44216
1 month ago
0-0
0 seconds
16316 mans0954
author:mans0954
feat(Analysis/Normed/Module/WeakDual): Banach Dieudonné Lemma WiP attempt to prove a lemma used in the proof of Banach Dieudonné Theorem Current proof is extremely scrappy. References: - Bourbaki TVS IV.24 - Conway, A course in Functional Analysis, 12.1 - Schaefer, p151 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-analysis WIP 390/3 Mathlib/Analysis/LocallyConvex/AbsConvex.lean,Mathlib/Analysis/LocallyConvex/Polar.lean,Mathlib/Analysis/Normed/Module/Dual.lean,Mathlib/Analysis/Normed/Module/WeakDual.lean,Mathlib/Topology/UniformSpace/Cauchy.lean 5 n/a ['github-actions'] nobody
37-44053
1 month ago
unknown
unknown
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$
48/24 Mathlib/Topology/Algebra/Module/FiniteDimension.lean,Mathlib/Topology/Algebra/Module/ModuleTopology.lean 2 5 ['erdOne', 'github-actions', 'matthewjasper'] nobody
37-13321
1 month ago
37-30391
1 month ago
38-85090
38 days
24574 JovanGerb
author:JovanGerb
chore(Order/Notation): check for pp options in `delabSup` The sup/inf delaborator shouldn't run when the user sets `pp.explicit true` or `pp.notation false`. This PR also removes my "-- TODO(Jovan): remove" edit: apparently, the fix in core wasn't fully successful. There still isn't support for adding/storing the localInstance inside `PPContext` or `MessageDataContext`. So we need that, or we need to extract the local instances anyways. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order 8/12 Mathlib/Order/Notation.lean 1 1 ['github-actions'] nobody
36-65896
1 month ago
37-270
1 month ago
37-320
37 days
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
36-59820
1 month ago
105-61462
3 months ago
105-61587
105 days
15213 adomani
author:adomani
dev: add Mathlib.Tactic.Linter.ForallIntro --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-linter WIP 608/0 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter.lean,Mathlib/Tactic/Linter/ForallIntro.lean,MathlibTest/ForallIntro.lean 5 4 ['adomani', 'github-actions', 'grunweg'] nobody
36-34563
1 month ago
36-34570
1 month ago
0-0
0 seconds
22488 smmercuri
author:smmercuri
fix: lower priority for `UniformSpace.Completion.instSMul` Following the introduction of the `WithVal` type synonym in #22055 the following instance takes a long time to synthesise in FLT, and times out in the default heartbeats ```lean import Mathlib namespace IsDedekindDomain.HeightOneSpectrum variable (A K : Type*) [CommRing A] [Field K] [Algebra A K] [IsFractionRing A K] [IsDedekindDomain A] (v : HeightOneSpectrum A) #synth SMul (v.adicCompletionIntegers K) (v.adicCompletion K) ``` The issue is that `UniformSpace.Completion.instSMul (v.adicCompletionIntegers K) (v.adicCompletion K)` now fires during the start of instance search (because we now have `UniformSpace (WithVal (v.valuation K))` whereas previously this would be `UniformSpace K`, which was not automatic), and this takes a long time to fail (leading to ~1400 entries in the trace). The first few lines of the new trace is ```lean [Meta.synthInstance] [5.512418] ✅️ SMul (↥(adicCompletionIntegers K v)) (adicCompletion K v) ▼ [] [0.000118] new goal SMul (↥(adicCompletionIntegers K v)) (adicCompletion K v) ▶ [] [0.000537] ✅️ apply UniformSpace.Completion.instSMul to SMul (↥(adicCompletionIntegers K v)) (adicCompletion K v) ▶ [] [0.004411] ✅️ apply @WithVal.instSMul to SMul (↥(adicCompletionIntegers K v)) (WithVal (valuation K v)) ▶ [] [0.000765] ❌️ apply @GradedMonoid.GradeZero.smul to SMul (↥(adicCompletionIntegers K v)) K ▶ [] [0.000378] ✅️ apply @Algebra.toSMul to SMul (↥(adicCompletionIntegers K v)) K ▶ ... [] 1339 more entries... ▶ ``` Lowering the priority of `UniformSpace.Completion.instSMul` fixes this particular issue, leading to a trace that matches that seen prior to the introduction of `WithVal`: ```lean [Meta.synthInstance] [0.016405] ✅️ SMul (↥(adicCompletionIntegers K v)) (adicCompletion K v) ▼ [] [0.000119] new goal SMul (↥(adicCompletionIntegers K v)) (adicCompletion K v) ▶ [] [0.000491] ❌️ apply @GradedMonoid.GradeZero.smul to SMul (↥(adicCompletionIntegers K v)) (adicCompletion K v) ▶ [] [0.000403] ✅️ apply @Algebra.toSMul to SMul (↥(adicCompletionIntegers K v)) (adicCompletion K v) ▶ [] [0.000134] ❌️ apply inst✝⁴ to Algebra (↥(adicCompletionIntegers K v)) (adicCompletion K v) ▶ [] [0.000093] ❌️ apply inst✝⁵ to Algebra (↥(adicCompletionIntegers K v)) (adicCompletion K v) ▶ [] [0.000077] ❌️ apply inst✝⁷ to Algebra (↥(adicCompletionIntegers K v)) (adicCompletion K v) ▶ [] [0.000082] ❌️ apply inst✝⁹ to Algebra (↥(adicCompletionIntegers K v)) (adicCompletion K v) ▶ [] [0.000075] ❌️ apply inst✝¹² to Algebra (↥(adicCompletionIntegers K v)) (adicCompletion K v) ▶ [] [0.000220] ❌️ apply Algebra.id to Algebra (↥(adicCompletionIntegers K v)) (adicCompletion K v) ▶ [] [0.001015] ✅️ apply @ValuationSubring.instAlgebraSubtypeMem to Algebra (↥(adicCompletionIntegers K v)) (adicCompletion K v) ▶ [resume] [0.000038] propagating Algebra (↥(adicCompletionIntegers K v)) (adicCompletion K v) to subgoal Algebra (↥(adicCompletionIntegers K v)) (adicCompletion K v) of SMul (↥(adicCompletionIntegers K v)) (adicCompletion K v) ▶ [check] [0.013358] ✅️ Algebra.toSMul [] result Algebra.toSMul ``` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) FLT t-topology awaiting-author 1/1 Mathlib/Topology/Algebra/UniformMulAction.lean 1 10 ['github-actions', 'leanprover-bot', 'smmercuri', 'urkud'] nobody
36-28000
1 month ago
42-56552
1 month ago
55-70108
55 days
15161 adomani
author:adomani
feat(Linter): flag `intros x y` which can be replaced by `intro x y` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-linter WIP 78/1 Mathlib/Tactic/Linter/Lint.lean,test/Lint.lean 2 4 ['adomani', 'github-actions', 'grunweg'] nobody
35-85468
1 month ago
36-33682
1 month ago
0-0
0 seconds
24620 mattrobball
author:mattrobball
chore(CategoryTheory.Basic): change `aesop_cat`'s intro transparency level to `instances` from `default` Let's see if this helps much. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 93/88 Mathlib/Algebra/Homology/HomologicalComplex.lean,Mathlib/Algebra/Homology/Homotopy.lean,Mathlib/Algebra/Homology/ShortComplex/Preadditive.lean,Mathlib/Algebra/Homology/Single.lean,Mathlib/CategoryTheory/Abelian/GrothendieckCategory/ModuleEmbedding/GabrielPopescu.lean,Mathlib/CategoryTheory/Adjunction/Comma.lean,Mathlib/CategoryTheory/Adjunction/Mates.lean,Mathlib/CategoryTheory/Bicategory/LocallyDiscrete.lean,Mathlib/CategoryTheory/Category/Basic.lean,Mathlib/CategoryTheory/Category/GaloisConnection.lean,Mathlib/CategoryTheory/CodiscreteCategory.lean,Mathlib/CategoryTheory/CommSq.lean,Mathlib/CategoryTheory/Comma/Over/Pullback.lean,Mathlib/CategoryTheory/Discrete/Basic.lean,Mathlib/CategoryTheory/EssentiallySmall.lean,Mathlib/CategoryTheory/FintypeCat.lean,Mathlib/CategoryTheory/Functor/EpiMono.lean,Mathlib/CategoryTheory/Functor/FullyFaithful.lean,Mathlib/CategoryTheory/Functor/KanExtension/Basic.lean,Mathlib/CategoryTheory/HomCongr.lean,Mathlib/CategoryTheory/Iso.lean,Mathlib/CategoryTheory/LiftingProperties/Adjunction.lean,Mathlib/CategoryTheory/Limits/ConeCategory.lean,Mathlib/CategoryTheory/Limits/HasLimits.lean,Mathlib/CategoryTheory/Limits/IsLimit.lean,Mathlib/CategoryTheory/Limits/Preserves/Shapes/Terminal.lean,Mathlib/CategoryTheory/Limits/Shapes/ZeroMorphisms.lean,Mathlib/CategoryTheory/MorphismProperty/OverAdjunction.lean,Mathlib/CategoryTheory/Preadditive/Opposite.lean,Mathlib/CategoryTheory/SingleObj.lean,Mathlib/Topology/Sheaves/Sheaf.lean 31 7 ['github-actions', 'leanprover-bot', 'mattrobball'] nobody
34-82871
1 month ago
35-1477
1 month ago
0-0
0 seconds
15649 TpmKranz
author:TpmKranz
feat(Computability): introduce Generalised NFA as bridge to Regular Expression Lays the groundwork for a proof of equivalence of NFA and RE, w.r.t. described language. Actual connection to NFA comes later, after the groundwork for the opposite direction has been laid. Second chunk of #12648 --- - [x] depends on: #15647 [Data.FinEnum.Option unchanged since then] [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-zulip t-computability new-contributor awaiting-author 298/0 Mathlib.lean,Mathlib/Computability/GNFA.lean,Mathlib/Computability/Language.lean,Mathlib/Computability/RegularExpressions.lean,docs/references.bib 5 6 ['github-actions', 'mathlib4-dependent-issues-bot', 'meithecatte', 'trivial1711'] nobody
34-77905
1 month ago
34-77914
1 month ago
23-54870
23 days
20648 anthonyde
author:anthonyde
feat: formalize regular expression -> εNFA The file `Computability/RegularExpressionsToEpsilonNFA.lean` contains a formal definition of Thompson's method for constructing an `εNFA` from a `RegularExpression` and a proof of its correctness. --- - [x] depends on: #20644 - [x] depends on: #20645 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-zulip t-computability new-contributor 490/0 Mathlib.lean,Mathlib/Computability/RegularExpressionsToEpsilonNFA.lean,docs/references.bib 3 5 ['github-actions', 'mathlib4-dependent-issues-bot', 'meithecatte', 'qawbecrdtey'] nobody
34-77216
1 month ago
34-77851
1 month ago
75-77754
75 days
22954 eric-wieser
author:eric-wieser
feat(RingTheory/Congruence/Hom): copy from GroupTheory This was motivated in review of #22355, but I no longer recall why. Either way, this captures a definition that was inlined in a later file. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
214/16 Mathlib/Algebra/RingQuot.lean,Mathlib/GroupTheory/Congruence/Hom.lean,Mathlib/RingTheory/Congruence/Defs.lean,Mathlib/RingTheory/Congruence/Hom.lean,Mathlib/RingTheory/TwoSidedIdeal/Kernel.lean 5 1 ['github-actions'] nobody
34-70531
1 month ago
86-26537
2 months ago
86-26580
86 days
23220 mattrobball
author:mattrobball
refactor(Module.LinearMap.Defs): make `SemilinearMapClass` extend `AddMonoidHomClass` Currently `SemilinearMapClass` extends `AddHomClass`. As both `SemilinearMapClass.toAddHomClass` and `AddMonoidHomClass.toAddHomClass` are projections, they have the same priority. With `SemilinearMapClass` declared later, it wins causing expensive failed searches in the algebraic hierarchy before `AddMonoidHomClass.toAddHomClass` is found. The current instance `SemilinearMapClass.toAddMonoidHomClass` has lower priority so we may need to downgrade the priority of the projection also. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra awaiting-author
label:t-algebra$
6/10 Mathlib/Algebra/Module/LinearMap/Defs.lean 1 9 ['eric-wieser', 'github-actions', 'leanprover-bot', 'mattrobball'] nobody
33-79351
1 month ago
33-79351
1 month ago
45-6308
45 days
24633 robin-carlier
author:robin-carlier
feat(Tactic/CategoryTheory): bicategory extension for `rotate_isos` This PR registers some lemmas to the `rotate_isos` tactic so that it applies in bicategorical contexts. For instance, if `α : g ⟶ h` is an invertible 2-cells, the term `f ◁ α ` is also recognized as invertible, with inverse `f ◁ α' `, where `α'` is the expression for the inverse constructed by the tactic. Without this extension, the tactic would only construct the generic `inv (f ◁ α)` as inverse for this term. --- - [ ] depends on: #24454 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory t-meta blocked-by-other-PR 1206/0 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/CategoryTheory/RotateIsos/Bicategory.lean,Mathlib/Tactic/CategoryTheory/RotateIsos/Cancelable.lean,Mathlib/Tactic/CategoryTheory/RotateIsos/Core.lean,Mathlib/Tactic/CategoryTheory/RotateIsos/Lemmas.lean,MathlibTest/CategoryTheory/RotateIsos.lean,scripts/noshake.json 8 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
33-44679
1 month ago
33-44679
1 month ago
0-945
15 minutes
24634 robin-carlier
author:robin-carlier
feat(Tactic/CategoryTheory): monoidal extension of `rotate_isos` This PR registers some lemmas to the `rotate_isos` tactic so that it applies in monoidal contexts. For instance, if α : y ⟶ z is an invertible morphism, the term x ◁ α is also recognized as invertible, with inverse x ◁ α' , where α' is the expression for the inverse constructed by the tactic. Without this extension, the tactic would only construct the generic inv (x ◁ α) as inverse for this term. We also take care of terms of the form `f ⊗ g` --- - [ ] depends on: #24454 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory t-meta blocked-by-other-PR 1362/0 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/CategoryTheory/RotateIsos/Cancelable.lean,Mathlib/Tactic/CategoryTheory/RotateIsos/Core.lean,Mathlib/Tactic/CategoryTheory/RotateIsos/Lemmas.lean,Mathlib/Tactic/CategoryTheory/RotateIsos/Monoidal.lean,MathlibTest/CategoryTheory/RotateIsos.lean,scripts/noshake.json 8 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
33-44667
1 month ago
33-44667
1 month ago
0-689
11 minutes
24650 robin-carlier
author:robin-carlier
feat(Tactic/CategoryTheory): whiskering lemmas for `rotate_isos` This PR extends the base set of terms recognized by the `rotate_isos` tactic to include terms of the form `whiskerLeft F f`, `isoWhiskerLeft F e`, and `NatTrans.hcomp`/ `NatIso.hcomp`. --- - [ ] depends on: #24454 Technically, it could depend solely on #24506, but there’s not much point getting this merged if the base tactic is not there. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta blocked-by-other-PR 1365/0 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/CategoryTheory/RotateIsos/Cancelable.lean,Mathlib/Tactic/CategoryTheory/RotateIsos/Core.lean,Mathlib/Tactic/CategoryTheory/RotateIsos/Lemmas.lean,MathlibTest/CategoryTheory/RotateIsos.lean,scripts/noshake.json 7 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
33-43388
1 month ago
33-43391
1 month ago
0-1022
17 minutes
24361 Hagb
author:Hagb
feat(Data/Finsupp/MonomialOrder): `0 ≤ a` where `a : m.syn` `simp` would be able to solve it. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data new-contributor easy 3/0 Mathlib/Data/Finsupp/MonomialOrder.lean 1 1 ['github-actions'] nobody
33-42488
1 month ago
33-42488
1 month ago
45-44165
45 days
24665 Komyyy
author:Komyyy
feat(Mathlib/Topology/Metrizable/Uniformity): every uniform space is generated by a family of pseudometrics --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology WIP 54/0 Mathlib/Topology/Metrizable/Uniformity.lean 1 1 ['github-actions'] nobody
33-1725
1 month ago
33-1725
1 month ago
0-1
1 second
24667 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). --- - [ ] depends on: #24321 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory blocked-by-other-PR 461/3 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', 'mathlib4-dependent-issues-bot'] nobody
32-78898
1 month ago
32-79449
1 month ago
0-235
3 minutes
24668 robertmaxton42
author:robertmaxton42
feat(LinearAlgebra): add inductive principle for the free product of algebras * Add `FreeProduct.inductionOn` and `.asPowers.inductionOn`. - [ ] depends on: #24532 --- * `simp↓` on `empty_rel'_bot`: the LHS is indeed not in simp-normal form, but `simp` can't solve the full lemma (if only because `Function.onFun` isn't marked `@[simp]`) and the actual simp-normal form of `rel'` isn't terribly useful for humans. Since I do expect users to type `rel' R A` by hand, I claim this use of `simp↓` is justified. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra blocked-by-other-PR
label:t-algebra$
205/9 Mathlib/LinearAlgebra/FreeProduct/Basic.lean 1 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
32-76559
1 month ago
32-77452
1 month ago
0-333
5 minutes
16150 urkud
author:urkud
feat(Dynamics): Hopf decomposition Prove Hopf decomposition. - [ ] rewrite to work with the saturations right away, not with a wandering set. - [ ] generalize to an action of a countable group, use fundamental domains. --- - [ ] depends on: #16146 - [ ] depends on: #16126 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-dynamics t-measure-probability 212/0 Mathlib.lean,Mathlib/Dynamics/Ergodic/Dissipative.lean,Mathlib/MeasureTheory/MeasurableSpace/Basic.lean 3 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'urkud'] nobody
32-57141
1 month ago
269-48791
8 months ago
0-0
0 seconds
22464 adomani
author:adomani
feat(CI): declarations diff in Lean Rewrites the `declaration_diff` script in Lean. You can see the effect of the new script in the testing branch #22497. The new CI step runs in approximately 5mins, but is separate from the `build` step. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) CI 151/0 .github/workflows/PR_summary_lean.yml,scripts/README.md,scripts/declarations_diff.lean,scripts/declarations_diff_lean_shell_glue.sh 4 6 ['bryangingechen', 'github-actions', 'grunweg'] robertylewis
assignee:robertylewis
32-46758
1 month ago
97-11003
3 months ago
97-10992
97 days
24172 LessnessRandomness
author:LessnessRandomness
feat: specialize rational root theorem to usual rational numbers and integers Rational root theorem and integral root theorem - the special case for usual rational numbers and integers. --- new-contributor t-algebra
label:t-algebra$
123/0 Mathlib.lean,Mathlib/RingTheory/Polynomial/OfRationalNumbers/RationalRootTheorem.lean 2 2 ['github-actions', 'grunweg'] mariainesdff
assignee:mariainesdff
32-46491
1 month ago
52-14174
1 month ago
52-14228
52 days
22792 madvorak
author:madvorak
feat(Mathlib/Data/Fin/Pigeonhole): pigeonhole-like results for Fin Consider the following settings: ``` import Mathlib example (X Y : Type) [Fintype X] [Fintype Y] (f : X → Y) (hf : f.Injective) : Fintype.card X ≤ Fintype.card Y := by hint example (m n : ℕ) (f : Fin m → Fin n) (hf : f.Injective) : m ≤ n := by hint example (X Y : Type) [Fintype X] [Fintype Y] (f : X ↪ Y) : Fintype.card X ≤ Fintype.card Y := by hint example (m n : ℕ) (f : Fin m ↪ Fin n) : m ≤ n := by hint ``` The 1st and 3rd `hint` succeed, but the 2nd a 4th `hint` fail. The problem is obviously that `exact?` does not see through `Fintype.card (Fin n) = n` when searching for appropriate lemma. It may seem to not be a problem, as it will rarely derail experienced Mathlib users — after all, experienced Leaners usually go directly for the `Finset` or `Fintype` version. However, beginners frequently work with `Fin` and they will expect stuff like ``` theorem le_of_injective (f : Fin m → Fin n) (hf : f.Injective) : m ≤ n ``` to exist; therefore, when `hint` or `exact?` fails, it is a very unpleasant surprise. This PR addressed this issue; not to provide useful content for advanced users, but to make Mathlib more useful for beginners. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data 38/0 Mathlib.lean,Mathlib/Data/Fin/Pigeonhole.lean 2 1 ['github-actions'] ericrbg
assignee:ericrbg
32-26308
1 month ago
91-16059
2 months ago
91-16110
91 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
32-26230
1 month ago
52-85074
1 month ago
63-47491
63 days
23826 javra
author:javra
feat(CategoryTheory): linear categories as `ModuleCat R`-enriched categories --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-category-theory 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 2 ['github-actions', 'leanprover-community-bot-assistant'] TwoFX
assignee:TwoFX
32-26214
1 month ago
56-36648
1 month ago
56-36630
56 days
24054 plp127
author:plp127
feat(Topology): R1 spaces are quasisober This generalizes `T2Space.quasiSober` --- - [ ] depends on: #24098 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology 36/8 Mathlib/Topology/Separation/Basic.lean,Mathlib/Topology/Separation/Hausdorff.lean,Mathlib/Topology/Sober.lean 3 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'urkud'] urkud
assignee:urkud
32-19721
1 month ago
47-9884
1 month ago
48-19934
48 days
16553 grunweg
author:grunweg
WIP: tinkering with orientable manifolds - wait for Rida's PR to get merged - PR the "normed space" part separately - WIP: a linear isomorphism on a connected set is either orientation-preserving or orientation-preserving: this will require #8738, it seems - [ ] depends on: #16239 - [ ] depends on: #8738 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-differential-geometry blocked-by-other-PR WIP 287/0 Mathlib.lean,Mathlib/Geometry/Manifold/Instances/Sphere.lean,Mathlib/Geometry/Manifold/Orientable.lean 3 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
31-81043
1 month ago
270-43908
8 months ago
0-0
0 seconds
23213 mattrobball
author:mattrobball
chore(RingTheory.Derivation): add a `LinearMapClass` instance Often we want `simp` to call `map_zero` or `map_add` for a `Derivation`. To find the `ZeroHomClass` or `AddHomClass` instance necessary it starts to climb up the type class hierarchy including looking for a `LinearMapClass` instance which didn't exist. Consequently, sythesis would look in a lot of crazy places trying to summon ring structures on the module or on derivations itself. Here we add the missing `LinearMapClass` instance so that `simp` is more efficient. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra delegated
label:t-algebra$
5/3 Mathlib/RingTheory/Derivation/Basic.lean 1 8 ['github-actions', 'j-loreaux', 'leanprover-bot', 'mathlib-bors', 'mattrobball'] nobody
31-78563
1 month ago
31-78563
1 month ago
47-39026
47 days
23214 mattrobball
author:mattrobball
perf(Module.LinearMap.Defs): deprioritize projections to parents for `SemilinearMapClass` Trying to figure out if a given type has a `SemilinearMapClass` instance when all we want is an `AddHomClass` or a `MulActionSemiHomClass` can be quite expensive since there are multiple ways to crawl the algebraic hierarchy to generate `LinearMapClass` instances. If these fail, then they fail slowly. We deprioritize the projections from `SemilinearMapClass` to `AddHomClass` and `MulActionSemiHomClass` to make this one of the last choices. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra delegated
label:t-algebra$
6/0 Mathlib/Algebra/Module/LinearMap/Defs.lean 1 6 ['github-actions', 'j-loreaux', 'leanprover-bot', 'mathlib-bors', 'mattrobball'] nobody
31-78329
1 month ago
31-78329
1 month ago
47-32152
47 days
23678 plp127
author:plp127
feat: recursor for nonempty lists Adds `List.recNeNil` and `List.recOnNeNil` for motives that depend on the list being nonempty. Taken from [Zulip](https://leanprover.zulipchat.com/#narrow/channel/217875-Is-there-code-for-X.3F/topic/accessing.20the.20source.20case.20during.20induction/near/502101211). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data 40/0 Mathlib/Data/List/Induction.lean 1 6 ['eric-wieser', 'github-actions', 'plp127'] ericrbg
assignee:ericrbg
31-75873
1 month ago
66-2110
2 months ago
66-2161
66 days
23930 Vtec234
author:Vtec234
feat(Tactic): dependent rewriting 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 --- 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 706/0 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/DepRewrite.lean,MathlibTest/depRewrite.lean 4 1 ['github-actions'] adamtopaz
assignee:adamtopaz
31-75742
1 month ago
59-70313
1 month ago
59-70362
59 days
24155 eric-wieser
author:eric-wieser
feat: add a "rw_proc" for fin vectors This seems a little nicer than an elaborator, since it means I can use the default elaboration rules to handle my first few variables. Ideally there would be something like ```lean rw_procQ {A : Type u} {B : A -> Type v} (a : A) (b : B a) : b = ?rhs => do /-- Context: u v : Level A : Q(Type u) B : Q($A -> Type v) a : Q($A) b : Q($B $a) rhs : Q($B $a) -- metavariable to assign |- MetaM Q($b = ?rhs) -/ ``` or ```lean rw_proc {A : Type u} {B : A -> Type v} (a : A) (b : B a) : b = ?rhs => do /-- Context: u v : Level A B a b : Expr rhs : MVarId |- MetaM Expr -/ ``` which would generate the code I wrote here --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data RFC t-meta awaiting-author 27/2 Mathlib/Data/Fin/Tuple/Reflection.lean 1 2 ['github-actions', 'urkud'] nobody
31-75706
1 month ago
31-75706
1 month ago
20-83091
20 days
24637 michaellee94
author:michaellee94
feat(Analysis/ODE/MaximalSolution): Existence of maximal solutions for ODE meeting Picard-Lindelöf conditions Add existence proof for maximal solution of ODE using Picard-Lindelöf and a uniqueness theorem using Grönwall's lemma. --- - [ ] depends on: #20704 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-analysis blocked-by-other-PR 746/1 Mathlib.lean,Mathlib/Analysis/ODE/MaximalSolution.lean,docs/undergrad.yaml 3 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'michaellee94'] nobody
31-70108
1 month ago
32-6233
1 month ago
2-10512
2 days
22314 shetzl
author:shetzl
feat: add leftmost derivations for context-free grammars Leftmost derivations are often easier to reason about than arbitrary derivations. This PR adds leftmost variants of Rewrites, Produces and Derives to the existing definition of context-free grammars and proves that a string of terminals can be derived iff it can be leftmost derived. Co-authored-by: Tobias Leichtfried --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-computability new-contributor awaiting-author 383/0 Mathlib.lean,Mathlib/Computability/LeftmostDerivation.lean 2 54 ['YaelDillies', 'github-actions', 'madvorak', 'shetzl'] YaelDillies
assignee:YaelDillies
31-36180
1 month ago
31-36180
1 month ago
72-3718
72 days
22196 xyzw12345
author:xyzw12345
feat: `lie_ring` tactic and `LieReduce` command In this PR, we implement a new tactic that reduces expressions in a `LieRing` to a normal form and checks whether they are equal, and a command which reduces the expression and displays the normal form. The implementation of this tactic imitates the `ring` tactic, using the `Qq` package to implement a specific reduction algorithm, following the theory of Hall sets and Lyndon words. A reference for the algorithm can be found at, for example, [here](https://personal.math.ubc.ca/~cass/research/pdf/Free.pdf). This project is the result of a workshop at Peking University, and @siddhartha-gadgil has helped us a lot on understanding the concepts in metaprogramming. Edit: The changes are reverted to a point where only `AtomM` is used. Co-authored-by: @Thmoas-Guan <2300010733@stu.pku.edu.cn> @yhtq <2100012990@stu.pku.edu.cn> @Blackfeather007 <2100017455@stu.pku.edu.cn> --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-meta 816/2 Mathlib.lean,Mathlib/Algebra/Lie/Derivation/AdjointAction.lean,Mathlib/Tactic.lean,Mathlib/Tactic/LieAlgebra/Basic.lean,Mathlib/Tactic/LieAlgebra/LieRingNF.lean,Mathlib/Util/AtomM.lean,MathlibTest/lie_ring.lean,scripts/noshake.json 8 16 ['bryangingechen', 'eric-wieser', 'faenuccio', 'github-actions', 'grunweg', 'ocfnash', 'siddhartha-gadgil', 'xyzw12345'] robertylewis
assignee:robertylewis
31-30093
1 month ago
106-61592
3 months ago
106-61583
106 days
24036 Louddy
author:Louddy
feat: add `HeightOneSpectrum.ofPrime` Add a definition relating elements of type `HeightOneSpectrum R` with the (nonzero) prime elements of the monoid with zero `Ideal R`. (Note the distinction between `Prime` and `Ideal.IsPrime`). The documentation string is inspired from [Ideal.prime_iff_isPrime](https://leanprover-community.github.io/mathlib4_docs/Mathlib/RingTheory/DedekindDomain/Ideal.html#Ideal.prime_iff_isPrime). This was discussed [#mathlib4 > Placing a definition in `DedekindDomain.Ideal` @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Placing.20a.20definition.20in.20.60DedekindDomain.2EIdeal.60/near/511647129). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra
label:t-algebra$
11/1 Mathlib/RingTheory/DedekindDomain/Ideal.lean 1 5 ['Louddy', 'Ruben-VandeVelde', 'github-actions'] Ruben-VandeVelde
assignee:Ruben-VandeVelde
31-28220
1 month ago
56-29490
1 month ago
56-29544
56 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 27 ['YaelDillies', 'b-mehta', 'eric-wieser', 'github-actions', 'kbuzzard', 'kmill', 'leanprover-community-mathlib4-bot'] kmill
assignee:kmill
31-28133
1 month ago
78-2807
2 months ago
126-22495
126 days
24710 chrisflav
author:chrisflav
chore(Data/Set): `tsum` version of `Set.encard_iUnion_of_finite` for non-finite types As requested here: https://github.com/leanprover-community/mathlib4/pull/23849#discussion_r2081070200 --- - [ ] depends on: #23849 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data blocked-by-other-PR 163/0 Mathlib.lean,Mathlib/Algebra/BigOperators/Finprod.lean,Mathlib/Data/Set/Card/Arithmetic.lean,Mathlib/Data/Set/Card/InfiniteArithmetic.lean,Mathlib/Data/Set/Finite/Lattice.lean,Mathlib/Topology/Algebra/InfiniteSum/Order.lean,Mathlib/Topology/Instances/ENat/Lemmas.lean 7 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
31-27778
1 month ago
31-27779
1 month ago
0-95
1 minute
22089 sgouezel
author:sgouezel
feat: composing a continuous multilinear map with continuous linear maps is analytic in both variables Also prove that the composition of continuously polynomial functions is continuously polynomial. --- - [x] depends on: #22102 - [x] depends on: #22789 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis 277/80 Mathlib/Analysis/Analytic/CPolynomial.lean,Mathlib/Analysis/Analytic/Composition.lean,Mathlib/Analysis/NormedSpace/Multilinear/Basic.lean,Mathlib/Data/Multiset/DershowitzManna.lean,Mathlib/Order/KrullDimension.lean 5 9 ['github-actions', 'grunweg', 'mathlib4-dependent-issues-bot', 'sgouezel', 'urkud'] loefflerd
assignee:loefflerd
31-23140
1 month ago
69-4593
2 months ago
107-57540
107 days
23320 Whysoserioushah
author:Whysoserioushah
feat(Mathlib/RingTheory/TwoSidedIdeal/SpanAsSum): span of set as finsum co-authored by: @jjaassoonn --- splited from [#23216](https://github.com/leanprover-community/mathlib4/pull/23216) following @eric-wieser advice [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
81/0 Mathlib.lean,Mathlib/RingTheory/TwoSidedIdeal/SpanAsSum.lean 2 43 ['Paul-Lez', 'Whysoserioushah', 'eric-wieser', 'github-actions', 'kbuzzard'] eric-wieser
assignee:eric-wieser
31-21018
1 month ago
75-73462
2 months ago
75-73506
75 days
21276 GabinKolly
author:GabinKolly
feat(ModelTheory/Substructures): define equivalences between equal substructures Define first-order equivalences between equal substructures, and prove related properties. --- This is some preparatory work for #18876 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-logic awaiting-author 62/0 Mathlib/ModelTheory/Substructures.lean 1 19 ['GabinKolly', 'YaelDillies', 'fpvandoorn', 'github-actions', 'grunweg'] nobody
31-11500
1 month ago
31-11500
1 month ago
46-55730
46 days
24727 dagurtomas
author:dagurtomas
feat(CategoryTheory): the universal property of localized monoidal categories This PR provides a monoidal structure on any functor out of a localized monoidal category whose precomposition with the localization functor is monoidal --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory WIP 457/0 Mathlib.lean,Mathlib/CategoryTheory/Localization/Bifunctor.lean,Mathlib/CategoryTheory/Localization/MonoidalFunctor.lean 3 1 ['github-actions'] nobody
31-1865
1 month ago
31-1865
1 month ago
0-2
2 seconds
23459 Timeroot
author:Timeroot
feat: Definition of `Clone` notations and typeclasses Definitions and notation typeclasses for #20051 --- [![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/Clone/Defs.lean 2 22 ['Timeroot', 'YaelDillies', 'dupuisf', 'eric-wieser', 'github-actions', 'urkud'] YaelDillies
assignee:YaelDillies
30-81075
30 days ago
63-17358
2 months ago
65-66460
65 days
23137 grunweg
author:grunweg
chore(Topology): some more fun_prop tagging --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology delegated 8/4 Mathlib/Dynamics/Flow.lean,Mathlib/Topology/Algebra/Monoid.lean 2 10 ['github-actions', 'grunweg', 'j-loreaux', 'mathlib-bors'] nobody
30-80778
30 days ago
30-80778
30 days ago
34-32727
34 days
24686 robin-carlier
author:robin-carlier
feat(CategoryTheory/Limits/Preserves/Bifunctor): construction of `PreservesColimit₂` instances Given a bifunctor `G : C₁ ⥤ C₂ ⥤ C` and two diagrams `K₁ : J₁ ⥤ C₁` and `K₂ : J₂ ⥤ C₂`, we show that if `C` has limits of shape `J₁`, `G` preserves the colimit of `K₁`, and `G` objectwise preserves colimits of `K₂`, then there is a `PreservesColimit₂ K₁ K₂ G` instance. We also show that if there is a `PreservesColimit₂ K₁ K₂ G` instance, then there is a `PreservesColimit₂ K₂ K₁ G.flip` instance as well. All results are dualised for limits. --- - [ ] depends on: #24685 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory blocked-by-other-PR 347/0 Mathlib.lean,Mathlib/CategoryTheory/Limits/Preserves/Bifunctor.lean 2 3 ['github-actions', 'joelriou', 'mathlib4-dependent-issues-bot'] nobody
30-80540
30 days ago
32-14612
1 month ago
0-498
8 minutes
24385 mans0954
author:mans0954
WIP: feature(Analysis/LocallyConvex/Prime): The prime map WiP: The "prime map" used in an investigation of the facial structure of closed unit balls in various Banach spaces in the work of Edwards and Rüttimann. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis WIP 125/0 Mathlib.lean,Mathlib/Analysis/LocallyConvex/Prime.lean 2 1 ['github-actions'] nobody
30-39667
30 days ago
44-34845
1 month ago
0-9
9 seconds
23162 mans0954
author:mans0954
feature(Analysis/SpecialFunctions/Complex/Log): exp_mul_I_injOn $e^{θi}$ is injective on `(-π, π]`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis WIP 11/0 Mathlib/Analysis/SpecialFunctions/Complex/CircleMap.lean 1 10 ['fbarroero', 'github-actions', 'j-loreaux', 'mans0954', 'urkud'] nobody
30-39578
30 days ago
43-33499
1 month ago
13-80660
13 days
24711 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/) 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 8 ['github-actions', 'joelriou', 'robin-carlier'] nobody
30-34702
30 days ago
30-34702
30 days ago
31-17992
31 days
20051 Timeroot
author:Timeroot
feat: `Clone` and some instances Defines clones (`Clone`). And there is a file, `Instances.lean`, that gives several most important examples of Clones. In particular, it has all of the clones (in an appropriately general form) that occur in [Post's Lattice](https://en.wikipedia.org/wiki/Post%27s_lattice), and [later proving](https://github.com/leanprover-community/mathlib4/pull/24744) the completeness of Post's Lattice is why I'm making this PR. (Edit: Used to also say "Defined operads (`Operad`), symmetric operads (`SymmOperad`), and clones ... There is a proof that all clones have a natural operad structure.". This has been scrapped.) --- - [x] depends on: #20133 [basics and notations] - [x] depends on: #20134 [permutations] - [x] depends on: #20138 [operad] - [x] depends on: #20141 [clone] - [ ] depends on: #23459 [defs] - [ ] depends on: #23460 [basic] [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra awaiting-author blocked-by-other-PR
label:t-algebra$
623/0 Mathlib.lean,Mathlib/Algebra/Clone/Basic.lean,Mathlib/Algebra/Clone/Defs.lean,Mathlib/Algebra/Clone/Instances.lean,Mathlib/Data/Fin/Basic.lean 5 32 ['Timeroot', 'YaelDillies', 'eric-wieser', 'github-actions', 'jcommelin', 'kbuzzard', 'kim-em', 'mathlib4-dependent-issues-bot', 'wmacmil'] nobody
30-20246
30 days ago
71-1973
2 months ago
43-16103
43 days
24351 eric-wieser
author:eric-wieser
feat: fderiv lemmas for `pow` This generalizes the lemmas about `fderiv fun x => f x ^ n` to work over arbitrary normed modules and algebras. Following the convention set by the lemmas about `fderiv` and `*`, we use `'`d names for the non-commutative variants. Moves: - `deriv_pow''` -> `deriv_pow` - `deriv_pow` -> `deriv_pow_field` - `derivWithin_pow'` -> `derivWithin_pow_field'` Deletions: - `deriv_pow'` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis 282/82 Mathlib.lean,Mathlib/Analysis/Calculus/Deriv/Polynomial.lean,Mathlib/Analysis/Calculus/Deriv/Pow.lean,Mathlib/Analysis/Calculus/FDeriv/Mul.lean,Mathlib/Analysis/Calculus/FDeriv/Pow.lean,Mathlib/Analysis/Calculus/Taylor.lean,Mathlib/Analysis/Complex/Angle.lean,Mathlib/Analysis/Convex/SpecificFunctions/Deriv.lean,Mathlib/NumberTheory/ModularForms/JacobiTheta/TwoVariable.lean 9 2 ['github-actions', 'leanprover-community-bot-assistant'] nobody
29-68522
29 days ago
29-68522
29 days ago
30-15569
30 days
22966 alreadydone
author:alreadydone
feat(RingTheory): degree of rational function field extension + `IsAlgebraic/IsIntegral R S` + `IsPushout R S R' S'` ⇒ `IsAlgebraic/IsIntegral R' S'` (for the "IsAlgebraic" version we currently need to assume `NoZeroDivisor R'` and `FaithfulSMul R R'` (i.e. `Injective (algebraMap R R')`) + `IsAlgebraic R S` + `IsFractionRing R R'` + `IsFractionRing S S'` ⇒ `IsPushout R S R' S'` (need to assume `FaithfulSMul R S` + `NonZeroDivisors S`) As consequences, we have `rank (f R) (f S) = rank R S` for `f = FractionRing (Polynomial ·)` or `FractionRing (MvPolynomial _ ·)` assuming `IsAlgebraic R S` + `IsDomain S` + `FaithfulSMul R S`. (For `f = Polynomial` or `MvPolynomial _`, `NoZeroDivisors R` is enough by #23095.) --- - [x] depends on: #23095 - [x] depends on: #23096 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
272/49 Mathlib/RingTheory/AdjoinRoot.lean,Mathlib/RingTheory/Algebraic/Basic.lean,Mathlib/RingTheory/Algebraic/Integral.lean,Mathlib/RingTheory/AlgebraicIndependent/AlgebraicClosure.lean,Mathlib/RingTheory/IntegralClosure/IsIntegralClosure/Basic.lean,Mathlib/RingTheory/TensorProduct/Basic.lean 6 11 ['Louddy', 'alreadydone', 'github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
29-64005
29 days ago
29-64974
29 days ago
47-35835
47 days
23594 YaelDillies
author:YaelDillies
refactor: merge `DomMulAct` and `DomAddAct` into `DomAct` This has several advantages: * Less API surface with a single definition instead of two * Better match the existing `ConjAct` type synonym * We get to use a better name for the multiplication by an element of the type synonym: Previously `dmaSMul`, now `domSMul`. and no inconvenient because the instances for `DomMulAct` and `DomAddAct` are by definition disjoint. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) file-removed t-algebra awaiting-CI
label:t-algebra$
328/326 Mathlib.lean,Mathlib/Algebra/Group/Translate.lean,Mathlib/Algebra/Module/CharacterModule.lean,Mathlib/Algebra/Module/Hom.lean,Mathlib/Algebra/Module/LinearMap/Basic.lean,Mathlib/Algebra/Module/LinearMap/Defs.lean,Mathlib/GroupTheory/GroupAction/DomAct/ActionHom.lean,Mathlib/GroupTheory/GroupAction/DomAct/Basic.lean,Mathlib/GroupTheory/Perm/Centralizer.lean,Mathlib/GroupTheory/Perm/DomAct.lean,Mathlib/MeasureTheory/Function/AEEqFun/DomAct.lean,Mathlib/MeasureTheory/Function/LpSpace/DomAct/Basic.lean,Mathlib/MeasureTheory/Function/LpSpace/DomAct/Continuous.lean,Mathlib/MeasureTheory/Group/MeasurableEquiv.lean,Mathlib/Topology/Algebra/Constructions/DomAct.lean,Mathlib/Topology/Algebra/Constructions/DomMulAct.lean 16 9 ['YaelDillies', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'urkud'] nobody
29-46999
29 days ago
29-46999
29 days ago
23-61670
23 days
24532 robertmaxton42
author:robertmaxton42
feat(LinearAlgebra/FreeProduct): fill out the `FreeProduct.asPowers` namespace * Replicate the existing API for `LinearAlgebra.FreeProduct` under `FreeProduct.asPowers`, for convenience when working primarily with the power algebra representation * Adds convenience lemmas for using the corresponding quotient relation `rel'` (used in the above). --- - [x] depends on: #24531 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
122/5 Mathlib/LinearAlgebra/FreeProduct/Basic.lean 1 25 ['YaelDillies', 'adomani', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'robertmaxton42'] nobody
29-41860
29 days ago
29-41912
29 days ago
30-3816
30 days
24008 meithecatte
author:meithecatte
chore(EpsilonNFA): replace manual lemmas with @[simps] --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-computability new-contributor awaiting-author 2/24 Mathlib/Computability/EpsilonNFA.lean 1 2 ['YaelDillies', 'github-actions', 'urkud'] nobody
29-37044
29 days ago
29-37044
29 days ago
27-52316
27 days
24571 Multramate
author:Multramate
refactor(AlgebraicGeometry/EllipticCurve/Affine/*): some minor changes --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebraic-geometry WIP 0/12 Mathlib.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Group.lean 2 n/a ['github-actions', 'leanprover-community-bot-assistant'] nobody
29-16827
29 days ago
unknown
unknown
24602 xyzw12345
author:xyzw12345
feat(LinearAlgebra/SymmetricAlgebra): IsSymmetricAlgebra This PR is a part of #21539, which separates out the part about `IsSymmetricAlgebra`. Co-authored-by: Raphael Douglas Giles @Raph-DG Co-authored-by: Zhixuan Dai <22300180006@m.fudan.edu.cn> Co-authored-by: Zhenyan Fu Co-authored-by: Yiming Fu - [ ] depends on: #21539 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
78/0 Mathlib/LinearAlgebra/SymmetricAlgebra/Basic.lean,Mathlib/LinearAlgebra/SymmetricAlgebra/Basis.lean 2 5 ['eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
29-11986
29 days ago
29-12238
29 days ago
29-14179
29 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
29-1394
29 days ago
29-7345
29 days ago
76-59566
76 days
21985 FernandoChu
author:FernandoChu
feat(CategoryTheory): the Grothendieck construction is prefibered Adds a `isPreFibered` instance for the Grothendieck construction. Co-authored-by: Christian Merten --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-category-theory awaiting-author 55/0 Mathlib/CategoryTheory/Bicategory/Functor/Pseudofunctor.lean,Mathlib/CategoryTheory/Bicategory/Grothendieck.lean 2 15 ['callesonne', 'chrisflav', 'github-actions'] nobody
28-82913
28 days ago
68-14237
2 months ago
8-4256
8 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 11 ['eric-wieser', 'github-actions', 'mathlib4-dependent-issues-bot', 'plp127', 'vihdzp'] nobody
28-72193
28 days ago
28-73125
28 days ago
94-73110
94 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
28-57787
28 days ago
28-57787
28 days ago
51-81907
51 days
22948 pelicanhere
author:pelicanhere
feat(Algebra/DirectSum): morphism of directsum decomposition Define morphism of directsum decomposition, which would be later used in defineing graded ring hom. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra
label:t-algebra$
83/0 Mathlib/Algebra/DirectSum/Decomposition.lean 1 9 ['eric-wieser', 'github-actions', 'pelicanhere'] eric-wieser
assignee:eric-wieser
28-41099
28 days ago
86-37917
2 months ago
86-37959
86 days
22531 vasnesterov
author:vasnesterov
feat(Analysis): radius of convergence for `FormalMultilinearSeries.compContinuousLinearMap` - Add basic lemmas `compContinuousLinearMap_id` and `compContinuousLinearMap_comp`. - Prove lower and upper bounds for the convergence radius of `f.compContinuousLinearMap`. - Prove `radius_compNeg`: the convergence radii of `f(x)` and `f(-x)` are equal. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis 137/11 Mathlib/Analysis/Analytic/Basic.lean,Mathlib/Analysis/Analytic/CPolynomial.lean,Mathlib/Analysis/Analytic/Constructions.lean,Mathlib/Analysis/Calculus/FormalMultilinearSeries.lean,scripts/noshake.json 5 7 ['github-actions', 'j-loreaux', 'vasnesterov'] nobody
28-7043
28 days ago
30-14317
30 days ago
95-9992
95 days
17627 hrmacbeth
author:hrmacbeth
feat: universal properties of vector bundle constructions Characterizations for the smoothness of maps into the total spaces of (1) the direct sum of two vector bundles; (2) the pullback of a vector bundle. This gap in the library was exposed by #17358. --- - [x] depends on: #22804 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-differential-geometry 311/9 Mathlib/Data/Bundle.lean,Mathlib/Geometry/Manifold/VectorBundle/Basic.lean,Mathlib/Geometry/Manifold/VectorBundle/Pullback.lean,Mathlib/Topology/FiberBundle/Constructions.lean 4 14 ['github-actions', 'grunweg', 'hrmacbeth', 'j-loreaux', 'mathlib4-dependent-issues-bot', 'sgouezel'] grunweg
assignee:grunweg
27-82562
27 days ago
81-30618
2 months ago
82-15074
82 days
24372 Hagb
author:Hagb
feat(Tactic/SimpIntro): add support for introducing non-propositions `simp_intro` would be able to introduce non-propositions. The previous `simp_intro` tactic cannot solve some statement that can be solved by applying `intro` and `simp` like `simp_intro`. For example, the following one can be solved like this ```lean example (r : Nat → Prop) : (∀ x, x > 0 → r x) → ∀ y z, y = 0 → z > y → r z := by simp intro hr try simp at hr -- does nothing try simp [hr] -- does nothing intro y z try simp [hr] -- does nothing intro hy try simp [hr] at hy -- does nothing simp [hr, hy] intro hyz try simp [hr, hy] at hyz simp [hr, hy, hyz] -- accomplish the goal successfully ``` while the previous `simp_intro` cannot introduce `y` and `z` here. ```lean example (r : Nat → Prop) : (∀ x, x > 0 → r x) → ∀ y z, y = 0 → z > y → r z := by /- the previous `simp_intro` fails with message: invalid 'simp', proposition expected Nat -/ simp_intro .. -- or `simp_intro hr y` example (r : Nat → Prop) : (∀ x, x > 0 → r x) → ∀ y z, y = 0 → z > y → r z := by -- unsolved simp_intro hr example (r : Nat → Prop) : (∀ x, x > 0 → r x) → ∀ y z, y = 0 → z > y → r z := by -- successfully solve the goal with the `simp_intro` in thie commit simp_intro .. -- or `simp_intro hr y z hy hz` ``` This commit makes it be able to introduce these kinds of hypotheses. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-meta 13/2 Mathlib/Tactic/SimpIntro.lean,MathlibTest/simp_intro.lean 2 1 ['github-actions'] kmill
assignee:kmill
27-81860
27 days ago
45-5392
1 month ago
45-5443
45 days
24395 rudynicolop
author:rudynicolop
feat(Data/List): list splitting definitions and lemmas Adds definitions and lemmas for obtaining all prefixes and suffixes of lists. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data new-contributor 143/2 Mathlib/Data/List/Perm/Lattice.lean,Mathlib/Data/List/TakeDrop.lean 2 1 ['github-actions'] ericrbg
assignee:ericrbg
27-81842
27 days ago
44-2869
1 month ago
44-2931
44 days
23497 chrisflav
author:chrisflav
chore(RingTheory/AdicCompletion/AsTensorProduct): golf using five lemma for modules --- - [x] depends on: #23496 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
30/81 Mathlib/RingTheory/AdicCompletion/AsTensorProduct.lean 1 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
27-75525
27 days ago
48-33482
1 month ago
48-34307
48 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
27-47902
27 days ago
27-56542
27 days ago
27-56596
27 days
24744 Timeroot
author:Timeroot
Post's lattice Draft PR for now so I can get CI checks. Eventually want to prove Post's Lattice --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) WIP 758/0 Mathlib.lean,Mathlib/Algebra/Clone/Basic.lean,Mathlib/Algebra/Clone/Defs.lean,Mathlib/Algebra/Clone/Instances.lean,Mathlib/Algebra/Clone/PostLattice.lean,Mathlib/Data/Fin/Basic.lean 6 1 ['github-actions'] nobody
27-43513
27 days ago
27-43513
27 days ago
0-0
0 seconds
23048 scholzhannah
author:scholzhannah
feat: PartialEquiv on closed sets restricts to closed map This PR shows that a PartialEquiv that is continuous on both source and target restricts to a homeomorphism. It then uses that to show that a PartialEquiv with closed source and target and which is continuous on both the source and target restricts to a closed map. --- See [this Zulip discussion](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Generalizing.20.60PartialHomeomorph.60.3F) that will probably mean that I close this PR. I need the latter statement to prove that one can transport a CW complex along a PartialEquiv. I had trouble finding a good spot for these statements; I hope this solution works. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-zulip t-topology 53/0 Mathlib.lean,Mathlib/Topology/PartialEquiv.lean 2 3 ['ADedecker', 'github-actions', 'scholzhannah'] ADedecker
assignee:ADedecker
27-15400
27 days ago
31-22176
1 month ago
51-86236
51 days
24793 tristan-f-r
author:tristan-f-r
feat: trace of unitarily similar matrices adds a theorem relating trace to unitarily similar matrices used in the easy direction of specht's theorem --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra awaiting-author
label:t-algebra$
7/0 Mathlib/LinearAlgebra/UnitaryGroup.lean 1 3 ['github-actions', 'j-loreaux', 'tristan-f-r'] nobody
27-14922
27 days ago
27-18456
27 days ago
1-55872
1 day
23177 faenuccio
author:faenuccio
feat: add order properties to WithZero types We add some order properties (mainly some `lt`) for types of the form `WithZero α`. Co-authored-by: María Inés de Frutos Fernández large-import t-order awaiting-CI 51/15 Mathlib/Algebra/GroupWithZero/Int.lean,Mathlib/Algebra/GroupWithZero/WithZero.lean,Mathlib/Algebra/Order/Group/Basic.lean,Mathlib/Algebra/Order/GroupWithZero/Canonical.lean,Mathlib/Algebra/Order/GroupWithZero/Unbundled/Basic.lean,Mathlib/Algebra/Order/Monoid/Unbundled/Pow.lean 6 43 ['Vierkantor', 'YaelDillies', 'faenuccio', 'github-actions'] nobody
27-10544
27 days ago
27-10545
27 days ago
5-22106
5 days
24752 MichaelStollBayreuth
author:MichaelStollBayreuth
perf(Data.Real.Sqrt): make Real.sqrt irreducible We try to see what happens if we make `Real.sqrt` irreducible. There are cases where this makes unification *very* significantly faster, compare [#mathlib4 > Coercion triggers timeout @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Coercion.20triggers.20timeout/near/517177117). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data 1/0 Mathlib/Data/Real/Sqrt.lean 1 18 ['MichaelStollBayreuth', 'eric-wieser', 'github-actions', 'leanprover-bot'] nobody
27-3829
27 days ago
29-17151
29 days ago
29-22628
29 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'] nobody
26-49284
26 days ago
26-49291
26 days ago
26-49435
26 days
24872 smmercuri
author:smmercuri
feat: `apply` and `coe` results for `UniformSpace.Completion.mapRingHom` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology 9/0 Mathlib/Topology/Algebra/UniformRing.lean 1 1 ['github-actions'] nobody
26-49063
26 days ago
26-49063
26 days ago
26-49111
26 days
24873 smmercuri
author:smmercuri
feat: `Subtype.map_ne` The restrictions to subtypes of two functions that never agree, also never agree. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data 7/0 Mathlib/Data/Subtype.lean 1 1 ['github-actions'] nobody
26-48723
26 days ago
26-48725
26 days ago
26-48774
26 days
24883 madvorak
author:madvorak
chore(Data/Matrix): `Matrix.submatrix` naming convention I'm suggesting this change for the following reasons: (1) managing expectations — `r_reindex` looks more like a propositional argument at first glance (2) the original naming does not do justice to its motivation — there is nothing called `r` and `c` here — it would need to be `row_reindex` and `col_reindex` or something like that (if we wanted to use the convention for naming constants even tho we are naming a variable here) --- Old version: https://github.com/leanprover-community/mathlib4/pull/24135 t-data 11/11 Mathlib/Data/Matrix/ConjTranspose.lean,Mathlib/Data/Matrix/Defs.lean 2 1 ['github-actions'] nobody
26-45358
26 days ago
26-45358
26 days ago
26-45348
26 days
23955 Louddy
author:Louddy
feat: Ideal.count_associates_eq Add variant of `UniqueFactorizationMonoid.count_normalizedFactors_eq` for associated Ideals. This is convenient when you need to talk about an element as `a₀ = x ^ n * a`. Note the file is slightly over the 1500 lines limit, I hope that is ok. 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/) new-contributor t-algebra
label:t-algebra$
35/1 Mathlib/RingTheory/DedekindDomain/Ideal.lean 1 7 ['Louddy', 'Ruben-VandeVelde', 'alreadydone', 'github-actions', 'grunweg'] kbuzzard
assignee:kbuzzard
26-44624
26 days ago
26-44624
26 days ago
53-45384
53 days
24892 Ruben-VandeVelde
author:Ruben-VandeVelde
fix: add missing simps projections for ContinuousAddEquiv --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology 1/0 Mathlib/Topology/Algebra/ContinuousMonoidHom.lean 1 1 ['github-actions'] nobody
26-36685
26 days ago
26-36687
26 days ago
26-36736
26 days
23999 YaelDillies
author:YaelDillies
feat: toric ideals From Toric Co-authored-by: Patrick Luo --- - [x] depends on: #22635 - [x] depends on: #24738 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) toric t-algebraic-geometry WIP 83/0 Mathlib.lean,Mathlib/AlgebraicGeometry/Toric/Ideal.lean 2 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
26-34559
26 days ago
26-35116
26 days ago
2-15562
2 days
24889 Kha
author:Kha
chore: do not include cache requests in build benchmark 5/2 scripts/bench/temci-config.run.yml 1 4 ['Kha', 'github-actions', 'leanprover-bot'] nobody
26-29277
26 days ago
26-39112
26 days ago
26-39095
26 days
22153 smmercuri
author:smmercuri
feat: weak approximation theorems for infinite places of a number field The number field $K$ is dense in $\prod_v (K, v)$ and in the infinite adele ring $\prod_v K_v$, where $v$ ranges over the infinite places, $(K, v)$ denotes $K$ equipped with the topology induced by $v$, and $K_v$ is the completion of $K$ at $v$. --- - [ ] depends on #22147 [![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$
543/2 Mathlib/Algebra/Order/AbsoluteValue/Basic.lean,Mathlib/Analysis/AbsoluteValue/Equivalence.lean,Mathlib/Analysis/Normed/Ring/WithAbs.lean,Mathlib/NumberTheory/NumberField/AdeleRing.lean,Mathlib/NumberTheory/NumberField/InfinitePlace/Basic.lean 5 1 ['github-actions'] nobody
26-25905
26 days ago
26-43208
26 days ago
37-66790
37 days
22142 smmercuri
author:smmercuri
feat: collections of non-trivial and pairwise inequivalent absolute values contain values that diverge around 1 The main result of this PR is that for a collection $v_1, ..., v_k$ of at least two non-trivial and pairwise inequivalent absolute values on a field $F$, there is an $a ∈ F$ such that $1 < v_1(a)$ while $v_j a < 1$ for all other $j ≠ 1$. --- - [ ] depends on: #22100 - [x] depends on: #22116 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-analysis blocked-by-other-PR
label:t-algebra$
380/1 Mathlib/Algebra/Order/AbsoluteValue/Basic.lean,Mathlib/Analysis/AbsoluteValue/Equivalence.lean,Mathlib/Analysis/Normed/Ring/WithAbs.lean,Mathlib/Data/Fin/Basic.lean 4 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
26-25753
26 days ago
52-85168
1 month ago
0-616
10 minutes
24618 b-mehta
author:b-mehta
feat(Analysis): add Schur inequality and variants Add Schur inequality and some of its common variants. TODO: - [x] add reference to source: https://www.cip.ifi.lmu.de/~grinberg/VornicuS.pdf - [ ] add other generalisations - [ ] move some of the lemmas elsewhere --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis WIP 145/0 Mathlib/Analysis/Convex/Schur.lean 1 16 ['b-mehta', 'eric-wieser', 'github-actions'] nobody
26-24577
26 days ago
35-4515
1 month ago
0-2
2 seconds
24311 YaelDillies
author:YaelDillies
chore: replace `Monoid.IsTorsionFree` with `IsMulTorsionFree` From Toric --- - [x] depends on: #24312 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) toric t-algebra
label:t-algebra$
63/29 Mathlib/Algebra/Group/Torsion.lean,Mathlib/Combinatorics/Additive/CauchyDavenport.lean,Mathlib/GroupTheory/Order/Min.lean,Mathlib/GroupTheory/Torsion.lean,Mathlib/Topology/Instances/ZMultiples.lean 5 5 ['YaelDillies', 'b-mehta', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
26-24432
26 days ago
26-24432
26 days ago
26-37762
26 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 15 ['YaelDillies', 'eric-wieser', 'github-actions', 'j-loreaux', 'leanprover-community-bot-assistant', 'mathlib-bors'] nobody
26-24175
26 days ago
26-24175
26 days ago
110-83611
110 days
23920 YaelDillies
author:YaelDillies
feat: entourage-separated sets Define a notion of separation of a set relative to an entourage. This will be used to unify metric and dynamical separation. From MiscYD and LeanAPAP --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology awaiting-author 61/0 Mathlib.lean,Mathlib/Topology/UniformSpace/Separated.lean 2 18 ['ADedecker', 'D-Thomine', 'YaelDillies', 'b-mehta', 'github-actions'] ADedecker
assignee:ADedecker
26-23406
26 days ago
26-23406
26 days ago
30-63355
30 days
23964 BoltonBailey
author:BoltonBailey
docs: Add documentation arbitrarily @mattrobball asked in the Mathlib Community meeting today what it would look like if we asked Claude code to give us improved documentation. I made this draft PR by selecting five declarations arbitrarily from `nolints.json` and asking Cursor to document them. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author documentation 52/14 Mathlib/Algebra/Homology/Homotopy.lean,Mathlib/Analysis/BoxIntegral/Partition/Filter.lean,Mathlib/Control/Monad/Cont.lean,Mathlib/Data/Stream/Defs.lean,Mathlib/LinearAlgebra/AffineSpace/AffineMap.lean 5 10 ['ADedecker', 'BoltonBailey', 'eric-wieser', 'github-actions', 'jcommelin', 'mattrobball'] nobody
25-49669
25 days ago
25-49669
25 days ago
33-13460
33 days
23881 YaelDillies
author:YaelDillies
feat: `ℝ≥0`-valued Lᵖ norm This is useful when inputting the Lp norm in places that expect a real number, like an exponent. From LeanAPAP --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-measure-probability awaiting-author 220/9 Mathlib.lean,Mathlib/MeasureTheory/Function/LpSeminorm/Defs.lean,Mathlib/MeasureTheory/Function/LpSeminorm/NNLpNorm.lean,Mathlib/MeasureTheory/Function/LpSeminorm/TriangleInequality.lean 4 18 ['YaelDillies', 'b-mehta', 'github-actions', 'leanprover-community-bot-assistant', 'sgouezel'] nobody
25-47917
25 days ago
26-36894
26 days ago
13-15316
13 days
24254 Louddy
author:Louddy
feat: valuation on RatFunc which is trivial on constants Given a valuation `v` on `RatFunc K` that is trivial on the constants `K`, the valuation on `RatFunc.X` determines to some degree the valuation on any `p : Polynomial K`. These are important in the context of Ostrowski's theorem for `RatFunc K`. Note that the condition that the valuation is trivial on constants is automatically fulfilled when `K` is finite. Co-authored-by: María Inés de Frutos Fernández <[mariaines.dff@gmail.com](mailto:mariaines.dff@gmail.com)> --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
66/0 Mathlib/FieldTheory/RatFunc/AsPolynomial.lean 1 29 ['Louddy', 'faenuccio', 'github-actions', 'mariainesdff'] nobody
25-33991
25 days ago
25-34043
25 days ago
27-34964
27 days
18379 oeb25
author:oeb25
feat(Topology/ENNReal): Add `ENNReal.tsum_biUnion` This adds infinite versions of `Finset.sum_biUnion` to `ENNReal`s. --- One notable difference from the `Finset` version is that for `tsum` we have two ways for selecting the summands: `∑' x : ⋃ i ∈ S` or `∑' x : ⋃ i, t i`. This PR adds both. I tried to extend this beyond `ENNReal`, but didn't find a clean way to do it. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-topology 34/0 Mathlib/Data/Set/Lattice.lean,Mathlib/Data/Set/Pairwise/Lattice.lean,Mathlib/Topology/Instances/ENNReal/Lemmas.lean 3 12 ['github-actions', 'grunweg', 'j-loreaux', 'oeb25'] nobody
25-33393
25 days ago
25-34406
25 days ago
127-82912
127 days
24912 YaelDillies
author:YaelDillies
feat: affine monoids Define affine monoids as finitely generated cancellative torsion-free commutative monoids and prove a few of their basic properties: * An affine monoid with no non-trivial unit is generated by its irreducible elements * An affine monoid embeds into `ℤⁿ` for some `n` * Let `M` be an affine monoid. If `R` is a domain, then so is `R[M]`. From Toric Co-authored-by: Patrick Luo --- - [ ] depends on: #24913 - [x] depends on: #24914 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) toric t-algebra blocked-by-other-PR
label:t-algebra$
199/3 Mathlib.lean,Mathlib/Algebra/AffineMonoid/Basic.lean,Mathlib/Algebra/AffineMonoid/Embedding.lean,Mathlib/Algebra/AffineMonoid/Irreducible.lean,Mathlib/Algebra/AffineMonoid/UniqueSums.lean,Mathlib/Algebra/Group/Irreducible/Defs.lean 6 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
25-22168
25 days ago
26-3587
26 days ago
0-479
7 minutes
24705 grunweg
author:grunweg
feat(workflows): automatically assign reviewers Once per day, automatically assign all proposed reviewers from the automatic assignment algorithm. --- See [the github documentation](https://docs.github.com/en/rest/issues/assignees?apiVersion=2022-11-28#add-assignees-to-an-issue) for the assignment syntax. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) CI help-wanted 42/0 .github/workflows/auto_assign_reviewers.yaml 1 13 ['adomani', 'bryangingechen', 'github-actions', 'grunweg'] bryangingechen
assignee:bryangingechen
25-17482
25 days ago
25-84554
25 days ago
2-20480
2 days
24730 YaelDillies
author:YaelDillies
feat(Bialgebra): group-like elements Define group-like elements in a bialgebra, ie units `a` such that `Δ a = a ⊗ₜ a`. We prove that group-like elements always form a group, and are linearly independent if the base ring is a domain. 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$
167/0 Mathlib.lean,Mathlib/RingTheory/Bialgebra/GroupLike.lean 2 18 ['YaelDillies', 'erdOne', 'eric-wieser', 'github-actions', 'leanprover-bot', 'mathlib4-dependent-issues-bot'] nobody
25-15390
25 days ago
29-79464
29 days ago
29-81020
29 days
24891 YaelDillies
author:YaelDillies
feat: `M ≃ₗ[R] (Fin (Module.finrank R M) → R)` for `M` a finite `R`-module From Toric --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) toric t-algebra
label:t-algebra$
13/3 Mathlib/LinearAlgebra/Dimension/Free.lean,Mathlib/LinearAlgebra/FreeModule/Basic.lean,Mathlib/LinearAlgebra/FreeModule/Finite/Basic.lean 3 9 ['YaelDillies', 'erdOne', 'eric-wieser', 'github-actions'] nobody
25-11279
25 days ago
26-21110
26 days ago
26-38032
26 days
22078 Louddy
author:Louddy
feat(SkewMonoidAlgebra): multiplication and algebraic instances # Multiplication and Algebraic Instances In this PR, we introduce the definition of the skewed convolution product on `SkewMonoidAlgebra k G`. Here, the product of two elements `f g : SkewMonoidAlgebra k G` is the finitely supported function whose value at `a` is the sum of `f x * (x • g y)` over all pairs `x, y` such that `x * y = a`. We also introduce the associated algebraic instances. ## Context This is the third part of a planned series of PRs aiming to formalise skew monoid algebras. The PRs are split to ease the review process. The moral sum of these planned PRs is #10541. The first and second part were #15878 and #19084. Co-authored-by: María Inés de Frutos Fernández <[mariaines.dff@gmail.com](mailto:mariaines.dff@gmail.com)> --- [![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$
453/45 Mathlib/Algebra/SkewMonoidAlgebra/Basic.lean 1 57 ['AntoineChambert-Loir', 'Louddy', 'github-actions', 'kbuzzard'] nobody
24-42459
24 days ago
26-39366
26 days ago
98-59896
98 days
24948 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/) t-combinatorics 91/0 Mathlib/Combinatorics/SimpleGraph/Bipartite.lean 1 1 ['github-actions'] nobody
24-40626
24 days ago
24-40631
24 days ago
24-40679
24 days
24838 RemyDegenne
author:RemyDegenne
feat(MeasureTheory): tightness of the range of a sequence * `isTightMeasureSet_range_iff_tendsto_limsup_measure_norm_gt`: in a proper normed group, the range of a sequence of measures `μ : ℕ → Measure E` is tight if and only if the function `r : ℝ ↦ limsup (fun n ↦ μ n {x | r < ‖x‖}) atTop` tends to `0` at infinity. * `isTightMeasureSet_range_iff_tendsto_limsup_inner`: in a finite-dimensional inner product space, the range of a sequence of measures `μ : ℕ → Measure E` is tight if and only if the function `r : ℝ ↦ limsup (fun n ↦ μ n {x | r < ‖⟪y, x⟫_𝕜‖}) atTop` tends to `0` at infinity for all `y`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-measure-probability awaiting-author 197/2 Mathlib/MeasureTheory/Measure/TightNormed.lean 1 7 ['RemyDegenne', 'github-actions', 'sgouezel'] nobody
24-32205
24 days ago
24-42642
24 days ago
2-82189
2 days
24957 eric-wieser
author:eric-wieser
feat: use ` binderNameHint` in sum_congr Zulip thread: [#new members > Choosing dummy variable inside summation @ 💬](https://leanprover.zulipchat.com/#narrow/channel/113489-new-members/topic/Choosing.20dummy.20variable.20inside.20summation/near/518492888) Co-authored-by: Joachim Breitner --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
23/16 Mathlib/Algebra/BigOperators/Expect.lean,Mathlib/Algebra/BigOperators/Group/Finset/Basic.lean,Mathlib/Analysis/BoxIntegral/Partition/Basic.lean,Mathlib/Data/Finset/Fold.lean,Mathlib/Data/Finset/Lattice/Fold.lean,Mathlib/Data/List/OfFn.lean,Mathlib/Data/Multiset/Count.lean,Mathlib/Data/Multiset/Filter.lean,Mathlib/Data/Multiset/MapFold.lean,Mathlib/Data/Option/Basic.lean,Mathlib/Data/Set/Image.lean,Mathlib/Data/Sym/Basic.lean,Mathlib/Data/Sym/Sym2.lean 13 1 ['github-actions'] nobody
24-23721
24 days ago
24-25171
24 days ago
24-25230
24 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 65/48 Mathlib/Analysis/Analytic/OfScalars.lean,Mathlib/Analysis/Oscillation.lean,Mathlib/Data/Finset/Lattice/Fold.lean,Mathlib/Data/Finset/Max.lean,Mathlib/LinearAlgebra/Eigenspace/Triangularizable.lean,Mathlib/MeasureTheory/Integral/Lebesgue/Countable.lean,Mathlib/MeasureTheory/Measure/LevyProkhorovMetric.lean,Mathlib/Order/Interval/Basic.lean,Mathlib/Order/Interval/Set/WithBotTop.lean,Mathlib/Order/WithBot.lean,Mathlib/Probability/Moments/Variance.lean,Mathlib/RingTheory/PowerBasis.lean,Mathlib/Topology/MetricSpace/Holder.lean,Mathlib/Topology/MetricSpace/HolderNorm.lean 14 20 ['YaelDillies', 'b-mehta', 'eric-wieser', 'github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'urkud'] nobody
23-44302
23 days ago
23-44323
23 days ago
73-36877
73 days
24967 vasnesterov
author:vasnesterov
perf(Topology/Metrizable): lower `IsCompletelyMetrizableSpace.MetrizableSpace` priority The priority of `IsCompletelyMetrizableSpace.MetrizableSpace` was set to 100, causing it to be applied before `EMetricSpace.metrizableSpace` and leading to wasted time trying to infer completeness. This PR sets it to 90. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology easy 1/1 Mathlib/Topology/Metrizable/CompletelyMetrizable.lean 1 4 ['github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot'] nobody
23-30787
23 days ago
23-69878
23 days ago
23-71889
23 days
23749 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 - [ ] depends on: #24967 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-analysis blocked-by-other-PR 48/1 Mathlib/Analysis/Analytic/ChangeOrigin.lean,Mathlib/Analysis/Calculus/IteratedDeriv/Lemmas.lean,Mathlib/Topology/Metrizable/CompletelyMetrizable.lean 3 4 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
23-29464
23 days ago
23-32732
23 days ago
0-220
3 minutes
22739 joelriou
author:joelriou
feat(CategoryTheory/Abelian): isomorphisms modulo a Serre class --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory 192/0 Mathlib.lean,Mathlib/CategoryTheory/Abelian/SerreClass/MorphismProperty.lean,Mathlib/CategoryTheory/Limits/Shapes/Equalizers.lean,Mathlib/CategoryTheory/Limits/Shapes/Kernels.lean,Mathlib/CategoryTheory/Preadditive/Basic.lean 5 7 ['TwoFX', 'erdOne', 'github-actions', 'joelriou'] nobody
23-22640
23 days ago
23-22640
23 days ago
81-8568
81 days
21162 smmercuri
author:smmercuri
feat: add `Valued.WithZeroMulInt.tendsto_zero_pow_of_le_neg_one` If `K` is a valued ring taking values in the multiplicative integers wth a zero adjoined, then `Valued.WithZeroMulInt.tendsto_zero_pow_of_le_neg_one` is the result that `x ^ n` tends to zero in this ring if `v x` is at most `-1` valued. --- - [x] depends on: #21160 - [x] depends on: #22055 - [ ] depends on: #24977 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra awaiting-author blocked-by-other-PR
label:t-algebra$
94/6 Mathlib.lean,Mathlib/Algebra/Group/Int/Defs.lean,Mathlib/Algebra/GroupWithZero/Int.lean,Mathlib/Algebra/GroupWithZero/WithZero.lean,Mathlib/Algebra/Order/GroupWithZero/Canonical.lean,Mathlib/RingTheory/Valuation/Discrete/Basic.lean,Mathlib/Topology/Algebra/Valued/WithZeroMulInt.lean 7 51 ['YaelDillies', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'smmercuri'] nobody
23-9796
23 days ago
23-9798
23 days ago
62-12390
62 days
5919 MithicSpirit
author:MithicSpirit
feat: implement orthogonality for AffineSubspace Define `AffineSubspace.orthogonal` and `AffineSubspace.IsOrtho`, as well as develop an API emulating that of `Submodule.orthogonal` and `Submodule.IsOrtho`, respectively. Additionally, provide some relevant lemmas exclusive to affine subspaces, which are mostly to do with the relationship between orthogonality and `AffineSubspace.Parallel`. Closes #5539 --- Still WIP as I need to add more docstrings as well as notations for the new definitions. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-analysis WIP help-wanted 287/0 Mathlib.lean,Mathlib/Analysis/InnerProductSpace/AffineSubspace.lean 2 6 ['MithicSpirit', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant'] MithicSpirit
assignee:MithicSpirit
23-7190
23 days ago
23-7208
23 days ago
0-0
0 seconds
10235 urkud
author:urkud
feat: add `Decidable`, `Fintype`, `Encodable` linters This PR ports the `decidableClassical`, `fintypeFinite` and `encodableCountable` linters from mathlib3: all three are environment linters which flag declarations that have a hypothesis `[Decidable p]` etc., but do not use the underlying assumption in this type. Restructuring the code can make the statement more general. The implementation is in fact quite general, and can easily adapt to include further types. PRs #17518 and #17519 are two examples of further such linters. --- Please don't fix the failures related to `HasFDerivWithinAt.pi`. Finiteness assumptions in these lemmas will be completely removed during porting to TVS. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-bench large-import t-linter t-meta awaiting-author 123/4 Mathlib.lean,Mathlib/Computability/Halting.lean,Mathlib/Computability/TuringMachine.lean,Mathlib/Data/Fintype/Quotient.lean,Mathlib/Logic/Basic.lean,Mathlib/Logic/Encodable/Basic.lean,Mathlib/NumberTheory/JacobiSum/Basic.lean,Mathlib/Order/Heyting/Regular.lean,Mathlib/Tactic.lean,Mathlib/Tactic/GeneralizeProofs.lean,Mathlib/Tactic/Linter/UnusedAssumptionInType.lean 11 n/a ['Command-Master', 'github-actions', 'grunweg', 'kmill', 'leanprover-bot', 'urkud'] nobody
23-5887
23 days ago
unknown
unknown
24533 robertmaxton42
author:robertmaxton42
feat (ULift): conjugation by ULift.up/down, misc cast/heq lemmas * Adds the convenience def `ULift.conj x := `down (f (up x))`, and corresponding basic lemmas * Adds lemmas showing that `ULift.up` and `.down` commute with casts and preserve `HEq`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data 31/0 Mathlib/Data/ULift.lean 1 14 ['eric-wieser', 'github-actions', 'robertmaxton42'] nobody
22-38855
22 days ago
38-38495
1 month ago
38-46410
38 days
24383 YaelDillies
author:YaelDillies
feat: distributive Haar characters of `ℝ` and `ℂ` Compute `distribHaarChar` in the case of the actions of `ℝˣ` on `ℝ` and of `ℂˣ` on `ℂ`. The file I'm moving was added two days ago and is not yet used in FLT. From FLT --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) FLT t-measure-probability awaiting-CI WIP 205/78 Mathlib.lean,Mathlib/Algebra/BigOperators/GroupWithZero/Action.lean,Mathlib/Algebra/Group/Action/BigOperators.lean,Mathlib/MeasureTheory/Measure/Haar/DistribChar/Basic.lean,Mathlib/MeasureTheory/Measure/Haar/DistribChar/Complex.lean,Mathlib/MeasureTheory/Measure/Haar/DistribChar/Real.lean,Mathlib/MeasureTheory/Measure/Lebesgue/Basic.lean,Mathlib/MeasureTheory/Measure/Lebesgue/EqHaar.lean 8 19 ['YaelDillies', 'github-actions', 'kbuzzard', 'leanprover-community-bot-assistant', 'sgouezel'] nobody
22-36243
22 days ago
27-47643
27 days ago
8-77637
8 days
24191 joelriou
author:joelriou
refactor(CategoryTheory): redefine triangulated subcategories using ObjectProperty --- - [x] depends on: #22574 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory 279/191 Mathlib/Algebra/Homology/DerivedCategory/Basic.lean,Mathlib/CategoryTheory/ObjectProperty/ContainsZero.lean,Mathlib/CategoryTheory/ObjectProperty/Shift.lean,Mathlib/CategoryTheory/Triangulated/HomologicalFunctor.lean,Mathlib/CategoryTheory/Triangulated/Subcategory.lean 5 5 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
22-30674
22 days ago
28-3496
28 days ago
46-67686
46 days
21032 joelriou
author:joelriou
feat(Order): bicartesian squares in lattices This PR introduces the notion of bicartesian square in lattices (and a more general "multicoequalizer" version in complete lattices). In the case of the lattice `Set X`, this will give respectively bicartesian squares (both pushout and pullback) and multicoequalizer diagrams in the category of sets. --- - [x] depends on: #22203 - [ ] depends on: #21026 - [x] depends on: #20988 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order t-category-theory blocked-by-other-PR WIP 195/0 Mathlib.lean,Mathlib/CategoryTheory/Limits/Shapes/MultiequalizerPullback.lean,Mathlib/Order/CompleteLattice/MulticoequalizerDiagram.lean 3 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
22-30425
22 days ago
61-25375
2 months ago
0-16
16 seconds
23364 joelriou
author:joelriou
refactor(CategoryTheory/Limits): colimits in Type --- - [x] depends on: #23346 - [ ] depends on: #23339 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory blocked-by-other-PR WIP 715/362 Mathlib.lean,Mathlib/Algebra/Category/Grp/Basic.lean,Mathlib/Algebra/Category/Grp/FilteredColimits.lean,Mathlib/Algebra/Category/ModuleCat/FilteredColimits.lean,Mathlib/Algebra/Category/MonCat/Basic.lean,Mathlib/Algebra/Category/MonCat/FilteredColimits.lean,Mathlib/Algebra/Category/Ring/Basic.lean,Mathlib/Algebra/Category/Ring/FilteredColimits.lean,Mathlib/CategoryTheory/Limits/Final.lean,Mathlib/CategoryTheory/Limits/FintypeCat.lean,Mathlib/CategoryTheory/Limits/IsConnected.lean,Mathlib/CategoryTheory/Limits/Preserves/Ulift.lean,Mathlib/CategoryTheory/Limits/Shapes/SingleObj.lean,Mathlib/CategoryTheory/Limits/Types/ColimitType.lean,Mathlib/CategoryTheory/Limits/Types/Colimits.lean,Mathlib/CategoryTheory/Limits/Types/Filtered.lean,Mathlib/CategoryTheory/Types.lean,Mathlib/Topology/Category/TopCat/Limits/Basic.lean 18 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
22-30226
22 days ago
22-30247
22 days ago
0-0
0 seconds
17469 joelriou
author:joelriou
feat(Algebra/ModuleCat/Differentials/Presheaf): the presheaf of relative differentials Given a functor `F : C ⥤ D`, presheaves of commutative rings `S`, `R` and a morphism `φ : S ⟶ F.op ⋙ R`, we show that derivations relative to `φ` are representable by a presheaf of `R`-modules. This is obtained by reducing to the case of absolute differentials. The construction shall allow to deduce the presheaf version of the cokernel sequence $$f^\star \Omega_{Y/S} ⟶ \Omega_{X/S} ⟶ \Omega_{X/Y} ⟶ 0$$ when `f : X ⟶ Y` and `g : Y ⟶ S` are morphisms of schemes. --- - [x] depends on: #17366 - [x] depends on: #19507 - [x] depends on: #17388 - [x] depends on: #16755 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-algebraic-geometry t-category-theory WIP 391/10 Mathlib/Algebra/Category/ModuleCat/Differentials/Presheaf.lean 1 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
22-28951
22 days ago
22-28970
22 days ago
0-530
8 minutes
22539 joelriou
author:joelriou
feat(Algebra/Homology): construction of left resolutions Given a fully faithful functor `ι : C ⥤ A` to an abelian category, we introduce a structure `Abelian.LeftResolutions ι` which gives a functor `F : A ⥤ C` and a natural epimorphism `π.app X : ι.obj (F.obj X) ⟶ X` for all `X : A`. This is used in order to construct a resolution functor `LeftResolutions.chainComplexFunctor : A ⥤ ChainComplex C ℕ`. This shall be used in order to derive the tensor product of modules and sheaves of modules. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory WIP 271/19 Mathlib.lean,Mathlib/Algebra/Homology/HomologicalComplex.lean,Mathlib/Algebra/Homology/LeftResolutions/Basic.lean,Mathlib/CategoryTheory/Limits/Shapes/Kernels.lean 4 1 ['github-actions'] nobody
22-28718
22 days ago
38-17536
1 month ago
59-17063
59 days
24993 robin-carlier
author:robin-carlier
feat(CategoryTheory/Monoidal/DayConvolution): left and right unitors for Day convolution Given a `DayConvolutionUnit U` a functor `F : C ⥤ V` and a Day convolution of `U` and `F`, we construct the left unitor isomorphism. `U ⊛ F ≅ F`. Similarly, given a Day convolution of `F` and `U`, we construct the right unitor. We characterize the isomorphisms, show their naturality, and show that the triangle identity is satisfied. --- - [ ] depends on: #24992 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory blocked-by-other-PR 954/0 Mathlib.lean,Mathlib/CategoryTheory/Functor/KanExtension/Basic.lean,Mathlib/CategoryTheory/Monoidal/DayConvolution.lean,Mathlib/CategoryTheory/Monoidal/ExternalProduct/Basic.lean,Mathlib/CategoryTheory/Monoidal/ExternalProduct/KanExtension.lean 5 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
22-19955
22 days ago
22-19957
22 days ago
0-173
2 minutes
24992 robin-carlier
author:robin-carlier
feat(CategoryTheory/Monoidal/DayConvolution): Associators and pentagon for Day Convolution Under some assumptions on the tensor product of a monoidal category `V`, we show that if three functors `F, G, H` are such that the relevant Day convolutions exist, then there is an associator isomorphism for day convolution. We characterize this isomorphism, and show it is natural. When all relevant Day convolutions exist, we show that the pentagon identity holds for these associators. --- - [ ] depends on: #24991 - [ ] depends on: #24989 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory blocked-by-other-PR 686/0 Mathlib.lean,Mathlib/CategoryTheory/Functor/KanExtension/Basic.lean,Mathlib/CategoryTheory/Monoidal/DayConvolution.lean,Mathlib/CategoryTheory/Monoidal/ExternalProduct/Basic.lean,Mathlib/CategoryTheory/Monoidal/ExternalProduct/KanExtension.lean 5 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
22-19954
22 days ago
22-19956
22 days ago
0-414
6 minutes
24991 robin-carlier
author:robin-carlier
feat(CategoryTheory/Monoidal): Day convolution of functors Given monoidal categories `C`,`V` and functors `F G : C ⥤ V`, we introduce a typeclass `[DayConvolution F G]` that bundles the data of a functor `F ⊛ G`, as well as the data required to exhibit `F ⊛ G` as a pointwise left Kan extension of `F ⊠ G` (the external product of `F` and `G`) along the tensor product of `C`. We give basic API around this class. We also define a class `DayConvolutionUnit U` which contains the data that `U` is pointwise left Kan extended from `fromPUnit (𝟙_ V)` along `fromPUnit (𝟙_ C)`. Again, we give basic API around this class. Properties like construction of associators and unitors isomorphisms (and the pentagon/triangle identities) will be the subject of subsequent PRs. --- - [ ] depends on: #24703 I opted to make `DayConvolution` a class to make assumptions on `C` and `V` minimal. Also, I realized that `C ⥤ V` already has a monoidal structure (given by pointwise tensor product), so trying to turn it into a monoidal category through Day convolution is probably pointless. What I intend to do instead is to define a typeclass `DayConvolutionMonoidalCategory A` that will extend `MonoidalCategory A`. This class will contain the data of a fully faithful functor `A ⥤ (C ⥤ V)`, and the data required to make it a "monoidal full subcategory" of `C ⥤ V`. This should allow us to register instances on type aliases for `C ⥤ V`, of course, there should be a constructor for this class that takes as input the embedding and existence of suitable pointwise extensions, and then turn it into a `DayConvolutionMonoidalCategory`. This is upcoming work [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory blocked-by-other-PR 309/0 Mathlib.lean,Mathlib/CategoryTheory/Functor/KanExtension/Basic.lean,Mathlib/CategoryTheory/Monoidal/DayConvolution.lean,Mathlib/CategoryTheory/Monoidal/ExternalProduct.lean 4 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
22-19953
22 days ago
22-19954
22 days ago
0-816
13 minutes
24989 robin-carlier
author:robin-carlier
feat(CategoryTheory/Monoidal/ExternalProduct): external product of left Kan extended functors Given a functor `H' : D' ⥤ V` to a monoidal category that is pointwise left Kan extended along `L : D ⥤ D'`, we show that for a functor `K : E ⥤ V` and under suitable preservations of colimits by the tensor product of `V`, the functor `H' ⊠ K : D' × E ⥤ V` is pointwise left Kan extended along `L.prod (𝟭 E)`. We show a similar statement for the functor `K ⊠ H'`. This property is crucial for proving properties of Day convolutions of functors from a monoidal category to `V`. --- - [ ] depends on: #24703 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory blocked-by-other-PR 244/0 Mathlib.lean,Mathlib/CategoryTheory/Monoidal/ExternalProduct/Basic.lean,Mathlib/CategoryTheory/Monoidal/ExternalProduct/KanExtension.lean 3 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
22-19951
22 days ago
22-19953
22 days ago
0-2653
44 minutes
24960 linesthatinterlace
author:linesthatinterlace
feat(Data/Finite/PermOf): Add an array-based implementation of finite permutations, `PermOf`. Implements `PermOf`, an array-based implementation of finite permutations/ --- As part of my PhD, I created this implementation. I have more to add to it, but I'm making this relatively small initial commit to exhibit the core definitions before I start building anything elaborate. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data 378/0 Mathlib.lean,Mathlib/Data/Finite/PermLT/Defs.lean,Mathlib/Data/Finite/PermLT/Group.lean,Mathlib/Data/Finite/PermLT/MulAction.lean 4 35 ['eric-wieser', 'github-actions', 'linesthatinterlace'] nobody
22-7695
22 days ago
24-19913
24 days ago
24-19968
24 days
22503 Kevew
author:Kevew
chore(Nat): Nat factorization multiplicity Ported lemmas from `Data/Nat/Multiplicity` to into a new file called `Data/Nat/Factorization/Multiplicity`, re-written in terms of `factorization`. --- - [x] depends on: #24576 - [ ] depends on: #25002 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-data new-contributor blocked-by-other-PR 327/101 Mathlib.lean,Mathlib/Data/Nat/Factorization/Basic.lean,Mathlib/Data/Nat/Factorization/LCM.lean,Mathlib/Data/Nat/Factorization/Multiplicity.lean,Mathlib/Data/Nat/Multiplicity.lean,Mathlib/GroupTheory/Exponent.lean,Mathlib/NumberTheory/Cyclotomic/PrimitiveRoots.lean,Mathlib/RingTheory/RootsOfUnity/PrimitiveRoots.lean 8 40 ['Kevew', 'Paul-Lez', 'YaelDillies', 'github-actions', 'grunweg', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] Kevew
assignee:Kevew
22-2003
22 days ago
25-44365
25 days ago
85-42249
85 days
24932 jkanschik
author:jkanschik
feat(Analysis/Calculus/VectorField): Implement product rule for liebrackets This adds lemmas for the product rule (or Leibniz rule) for Lie brackets on vector fields. These new lemmas are called `lieBracket_smul_left` and similar. To accomodate this, rename the existing lemmas `{m}lieBracket{Within}_smul_{left,right}` to `{m}lieBracket{Within}_const_smul_{left,right}`. An additional PR for the same functionality on manifolds is in preparation and would depend on this PR. This will become useful when introducing Lie derivatives or covariant derivatives in differential geometry. new-contributor t-differential-geometry awaiting-author 78/28 Mathlib/Analysis/Calculus/VectorField.lean,Mathlib/Geometry/Manifold/GroupLieAlgebra.lean,Mathlib/Geometry/Manifold/VectorField/LieBracket.lean 3 30 ['github-actions', 'grunweg', 'jkanschik', 'sgouezel'] nobody
22-715
22 days ago
23-30023
23 days ago
1-1522
1 day
24966 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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-differential-geometry 154/13 Mathlib/Geometry/Manifold/PartitionOfUnity.lean 1 3 ['github-actions', 'grunweg', 'michaellee94'] nobody
21-79963
21 days ago
23-17943
23 days ago
23-45496
23 days
19796 peakpoint
author:peakpoint
feat: L'Hopital's rule from within a convex set --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-analysis 190/19 Mathlib/Algebra/Polynomial/Module/Basic.lean,Mathlib/Analysis/Calculus/LHopital.lean,Mathlib/Analysis/Convex/Topology.lean,Mathlib/Geometry/Manifold/Instances/Real.lean,Mathlib/Order/Interval/Set/Basic.lean 5 14 ['RemyDegenne', 'github-actions', 'leanprover-community-bot-assistant', 'peakpoint', 'sgouezel'] sgouezel
assignee:sgouezel
21-79134
21 days ago
21-79134
21 days ago
55-29418
55 days
17458 urkud
author:urkud
refactor(Algebra/Group): make `IsUnit` a typeclass Also change some lemmas to assume `[IsUnit _]` instead of `[Invertible _]`. Motivated by potential non-defeq diamonds in #14986, see also [Zulip](https://leanprover.zulipchat.com/#narrow/stream/116395-maths/topic/Invertible.20and.20data) I no longer plan to merge this PR, but I'm going to cherry-pick some changes to a new PR before closing this one. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-zulip t-algebra
label:t-algebra$
82/72 Mathlib/Algebra/CharP/Invertible.lean,Mathlib/Algebra/Group/Invertible/Basic.lean,Mathlib/Algebra/Group/Units/Defs.lean,Mathlib/Algebra/GroupWithZero/Invertible.lean,Mathlib/Algebra/GroupWithZero/Units/Basic.lean,Mathlib/Algebra/Polynomial/Degree/Units.lean,Mathlib/Algebra/Polynomial/Splits.lean,Mathlib/Analysis/Convex/Segment.lean,Mathlib/Analysis/Normed/Affine/Isometry.lean,Mathlib/Analysis/Normed/Ring/Units.lean,Mathlib/CategoryTheory/Linear/Basic.lean,Mathlib/FieldTheory/Finite/Basic.lean,Mathlib/FieldTheory/Separable.lean,Mathlib/FieldTheory/SeparableDegree.lean,Mathlib/GroupTheory/Submonoid/Inverses.lean,Mathlib/LinearAlgebra/AffineSpace/AffineEquiv.lean,Mathlib/LinearAlgebra/AffineSpace/Combination.lean,Mathlib/LinearAlgebra/CliffordAlgebra/Contraction.lean,Mathlib/LinearAlgebra/CliffordAlgebra/Inversion.lean,Mathlib/LinearAlgebra/CliffordAlgebra/SpinGroup.lean,Mathlib/LinearAlgebra/Eigenspace/Minpoly.lean,Mathlib/NumberTheory/MulChar/Basic.lean,Mathlib/RingTheory/Localization/NumDen.lean,Mathlib/RingTheory/Polynomial/Content.lean,Mathlib/RingTheory/Polynomial/GaussLemma.lean,Mathlib/RingTheory/Valuation/Basic.lean 26 11 ['MichaelStollBayreuth', 'acmepjz', 'eric-wieser', 'github-actions', 'leanprover-bot', 'urkud'] nobody
21-63866
21 days ago
21-84293
21 days ago
0-66650
18 hours
24435 faenuccio
author:faenuccio
chore(RingTheory/Valuation/Discrete/Basic): add ordered Iso between Z_{m0} and the value group large-import t-order t-algebra WIP
label:t-algebra$
267/28 Mathlib/Algebra/GroupWithZero/Int.lean,Mathlib/Algebra/Order/Group/Cyclic.lean,Mathlib/RingTheory/Valuation/Discrete/Basic.lean 3 5 ['faenuccio', 'github-actions', 'leanprover-community-bot-assistant', 'mariainesdff'] nobody
21-28505
21 days ago
28-5843
28 days ago
0-3
3 seconds
21522 riccardobrasca
author:riccardobrasca
feat: add Mathlib.RingTheory.DedekindDomain.Instances We add a new file `Mathlib.RingTheory.DedekindDomain.Instances` containing various instances that are useful to work with the localization a prime of an extension of Dedekind domains. As a practical example we golf a tedious proof in `Mathlib.RingTheory.Ideal/Norm.RelNorm` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-algebra
label:t-algebra$
253/71 Mathlib.lean,Mathlib/RingTheory/DedekindDomain/Different.lean,Mathlib/RingTheory/DedekindDomain/Instances.lean,Mathlib/RingTheory/DedekindDomain/IntegralClosure.lean,Mathlib/RingTheory/Ideal/Norm/RelNorm.lean,Mathlib/RingTheory/IntegralClosure/IntegralRestrict.lean,Mathlib/RingTheory/Localization/AtPrime.lean,Mathlib/RingTheory/Localization/Basic.lean,Mathlib/RingTheory/Localization/LocalizationLocalization.lean,Mathlib/RingTheory/RingHom/Finite.lean,Mathlib/RingTheory/Trace/Quotient.lean 11 34 ['YaelDillies', 'erdOne', 'fpvandoorn', 'github-actions', 'riccardobrasca'] nobody
21-26828
21 days ago
26-26297
26 days ago
92-58869
92 days
24719 madvorak
author:madvorak
feat(LinearAlgebra/Matrix/NonsingularInverse): inverting `Matrix` inverts its `LinearEquiv` --- Discussion: https://leanprover.zulipchat.com/#narrow/channel/144837-PR-reviews/topic/.2324719.20cannot.20find.20home/with/517142655 t-algebra
label:t-algebra$
10/0 Mathlib/LinearAlgebra/Matrix/NonsingularInverse.lean 1 11 ['eric-wieser', 'github-actions', 'madvorak'] nobody
21-20152
21 days ago
29-24997
29 days ago
30-61226
30 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
21-9651
21 days ago
21-9775
21 days ago
21-13240
21 days
25036 Parcly-Taxel
author:Parcly-Taxel
feat: IMO 2001 Q4 IMO 131/4 Archive.lean,Archive/Imo/Imo2001Q4.lean,Mathlib/Logic/Equiv/Fin/Rotate.lean 3 1 ['github-actions'] nobody
20-51766
20 days ago
20-52508
20 days ago
20-52492
20 days
21624 sinhp
author:sinhp
feat(CategoryTheory): The (closed) monoidal structure on the product category of families of (closed) monoidal categories Given a family of closed monoidal categories, we show that the product of these categories is a closed monoidal category with the pointwise monoidal structure. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory awaiting-author 144/0 Mathlib.lean,Mathlib/CategoryTheory/Pi/Basic.lean,Mathlib/CategoryTheory/Pi/Monoidal.lean,Mathlib/CategoryTheory/Pi/MonoidalClosed.lean 4 19 ['TwoFX', 'YaelDillies', 'b-mehta', 'github-actions', 'jcommelin', 'sinhp'] nobody
20-45417
20 days ago
20-45417
20 days ago
54-54882
54 days
24855 euprunin
author:euprunin
feat: register more tactics for `hint` The following example shows test cases that `hint` now supports, which were unsupported prior to this PR: ``` import Mathlib -- The tactics registered in this PR register_hint compute_degree register_hint field_simp register_hint finiteness -- "hint" now correctly suggests "compute_degree" which closes the goal (no closing tactic suggested prior to this PR) open Polynomial in example : natDegree ((X + 1) : Nat[X]) ≤ 1 := by hint -- "hint" now correctly suggests "field_simp" which closes the goal (no closing tactic suggested prior to this PR) example (R : Type) (a b : R) [CommRing R] (u₁ : Rˣ) : a /ₚ u₁ + b /ₚ u₁ = (a + b) /ₚ u₁ := by hint -- "hint" now correctly suggests "finiteness" which closes the goal (no closing tactic suggested prior to this PR) example (a : ℝ) : (ENNReal.ofReal (1 + a ^ 2))⁻¹ < ⊤ := by hint ``` t-meta awaiting-author 15/0 Mathlib/Tactic/ComputeDegree.lean,Mathlib/Tactic/FieldSimp.lean,Mathlib/Tactic/Finiteness.lean 3 7 ['adomani', 'euprunin', 'github-actions', 'grunweg'] nobody
20-45388
20 days ago
20-45388
20 days ago
0-24945
6 hours
22151 alreadydone
author:alreadydone
feat(RingTheory): a semiprimary ring is Noetherian/Artinian iff its Jacobson radical is fg A key fact used is `Module.FG.smul`: if `I` is a two-sided ideal of `R` that is f.g. as a left ideal and `N` is a f.g. `R`-module, then `I • M` is also a f.g. `R`-module. Many lemmas about coprimality of ideals are also generalized to the noncommutative, two-sided setting. --- - [x] depends on: #21904 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
215/155 Mathlib/Algebra/Algebra/Operations.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Affine/Point.lean,Mathlib/RingTheory/Extension/Basic.lean,Mathlib/RingTheory/Finiteness/Basic.lean,Mathlib/RingTheory/Finiteness/Ideal.lean,Mathlib/RingTheory/HopkinsLevitzki.lean,Mathlib/RingTheory/Ideal/Maps.lean,Mathlib/RingTheory/Ideal/Operations.lean 8 7 ['alreadydone', 'github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
20-38962
20 days ago
20-39117
20 days ago
97-8246
97 days
20160 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/) t-data 69/0 Mathlib/Data/Seq/Seq.lean 1 3 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
20-37866
20 days ago
27-81161
27 days ago
27-81310
27 days
22631 Thmoas-Guan
author:Thmoas-Guan
feat(Algebra): define associated graded structure for abelian group In this PR we define the associated graded structure for abelian group when given a filtration and only give some basic lemmas about it. Further results would be given in #20913 --- - [x] depends on: #24071 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
155/0 Mathlib.lean,Mathlib/RingTheory/FilteredAlgebra/AssociatedGraded.lean 2 17 ['AntoineChambert-Loir', 'Thmoas-Guan', 'eric-wieser', 'github-actions', 'kbuzzard', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
20-35308
20 days ago
20-35328
20 days ago
94-79909
94 days
20913 Thmoas-Guan
author:Thmoas-Guan
feat(Algebra): Define the associated graded ring to filtered ring. Define the associated graded ring to a filtered ring. --- - [x] depends on: #20900 - [x] depends on: #22230 - [ ] depends on: #22631 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra blocked-by-other-PR
label:t-algebra$
442/0 Mathlib.lean,Mathlib/RingTheory/FilteredAlgebra/AssociatedGraded.lean 2 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
20-35139
20 days ago
20-35158
20 days ago
0-70480
19 hours
21806 Thmoas-Guan
author:Thmoas-Guan
feat(Algebra): associated graded algebra Define the associated graded algebra of a filtered algebra, constructed from a special case of associated graded ring. --- - [x] depends on: #20900 - [ ] depends on: #20913 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra blocked-by-other-PR WIP
label:t-algebra$
552/0 Mathlib.lean,Mathlib/RingTheory/FilteredAlgebra/AssociatedGraded.lean 2 n/a ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
20-35082
20 days ago
unknown
unknown
20940 Thmoas-Guan
author:Thmoas-Guan
feat(Algebra): Associated graded module Define the associated graded module to a filtered module. --- - [x] depends on: #20900 - [ ] depends on: #20913 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra blocked-by-other-PR WIP
label:t-algebra$
656/0 Mathlib.lean,Mathlib/RingTheory/FilteredAlgebra/AssociatedGraded.lean 2 n/a ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] Blackfeather007
assignee:Blackfeather007
20-34999
20 days ago
unknown
unknown
22632 Thmoas-Guan
author:Thmoas-Guan
feat(Algebra): define filtered add group hom In this file we define filtered hom and the corresponding associated graded hom for abelian groups. Co-authored-by: Huanyu Zheng @Yu-Misaka Co-authored-by: Yi Yuan @yuanyi-350 Co-authored-by: Weichen Jiao @AlbertJ-314 --- - [ ] depends on: #22631 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra blocked-by-other-PR
label:t-algebra$
378/0 Mathlib.lean,Mathlib/RingTheory/FilteredAlgebra/AssociatedGraded.lean,Mathlib/RingTheory/FilteredAlgebra/FilteredHom.lean 3 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
20-34810
20 days ago
20-34831
20 days ago
0-1204
20 minutes
22208 Thmoas-Guan
author:Thmoas-Guan
feat(Algebra):filtered ring hom In this PR, we define the filtered ring morphisms on rings and prove some basic properties of them. Co-authored-by: Huanyu Zheng @Yu-Misaka Co-authored-by: Yi Yuan @yuanyi-350 Co-authored-by: Weichen Jiao @AlbertJ-314 --- - [ ] depends on: #20913 - [ ] depends on: #22632 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra blocked-by-other-PR
label:t-algebra$
812/0 Mathlib.lean,Mathlib/RingTheory/FilteredAlgebra/AssociatedGraded.lean,Mathlib/RingTheory/FilteredAlgebra/FilteredHom.lean 3 n/a ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
20-34730
20 days ago
unknown
unknown
22454 Thmoas-Guan
author:Thmoas-Guan
feat(Algebra): define filtered algebra morphisms In this PR, we define the filtered algebra morphisms on algebras and prove some basic properties of them. --- - [ ] depends on: #21806 - [ ] depends on: #22208 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra blocked-by-other-PR WIP
label:t-algebra$
1039/0 Mathlib.lean,Mathlib/RingTheory/FilteredAlgebra/AssociatedGraded.lean,Mathlib/RingTheory/FilteredAlgebra/FilteredHom.lean 3 n/a ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
20-34659
20 days ago
unknown
unknown
22893 Thmoas-Guan
author:Thmoas-Guan
feat(Algebra): filtered module hom In this PR we defined the filtered semi-linear map for filtered module and the associated graded module hom. --- - [ ] depends on: #22208 - [ ] depends on: #20940 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra blocked-by-other-PR
label:t-algebra$
1187/0 Mathlib.lean,Mathlib/RingTheory/FilteredAlgebra/AssociatedGraded.lean,Mathlib/RingTheory/FilteredAlgebra/FilteredHom.lean 3 n/a ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
20-34612
20 days ago
unknown
unknown
22707 Thmoas-Guan
author:Thmoas-Guan
feat(Algebra): associated graded exact of exact and strict In this file, we define the concept of exhaustive filtrations. We also prove a AssociatedGradedRingHom sequence is exact iff each GradedPieceHom is exact. And when a sequence is strict exact, the corresponding AssociatedGradedRingHom sequence is also exact. Co-authored-by: Huanyu Zheng @Yu-Misaka Co-authored-by: Yi Yuan @yuanyi-350 Co-authored-by: Weichen Jiao @AlbertJ-314 --- - [ ] depends on: #22632 - [x] depends on: #22705 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra blocked-by-other-PR
label:t-algebra$
534/0 Mathlib.lean,Mathlib/RingTheory/FilteredAlgebra/AssociatedGraded.lean,Mathlib/RingTheory/FilteredAlgebra/Exactness.lean,Mathlib/RingTheory/FilteredAlgebra/FilteredHom.lean 4 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
20-34552
20 days ago
20-34573
20 days ago
0-464
7 minutes
22972 Thmoas-Guan
author:Thmoas-Guan
feat(Algebra): exact of associated graded exact We proved that a chain complex is exact if its associated graded complex is exact. Co-authored-by: Huanyu Zheng @Yu-Misaka Co-authored-by: Yi Yuan @yuanyi-350 Co-authored-by: Weichen Jiao @AlbertJ-314 --- - [ ] depends on: #22632 - [x] depends on: #22705 - [ ] depends on: #22707 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra blocked-by-other-PR
label:t-algebra$
729/0 Mathlib.lean,Mathlib/RingTheory/FilteredAlgebra/AssociatedGraded.lean,Mathlib/RingTheory/FilteredAlgebra/Exactness.lean,Mathlib/RingTheory/FilteredAlgebra/FilteredHom.lean 4 n/a ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
20-34488
20 days ago
unknown
unknown
24949 RemyDegenne
author:RemyDegenne
feat: tightness from convergence of characteristic functions If the characteristic functions of a sequence of measures `μ : ℕ → Measure E` on a finite dimensional inner product space converge pointwise to a function which is continuous at 0, then `{μ n | n}` is tight. --- - [ ] depends on: #24838 - [x] depends on: #24846 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-measure-probability blocked-by-other-PR WIP 352/2 Mathlib.lean,Mathlib/MeasureTheory/Measure/TightCharFun.lean,Mathlib/MeasureTheory/Measure/TightNormed.lean 3 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
20-29663
20 days ago
20-29679
20 days ago
0-2
2 seconds
25044 alreadydone
author:alreadydone
feat(Topology/Algebra): `Homeomorph` version of `unitsEquivNeZero` also add `Topology.IsEmbedding.homeomorphImage`: a set is homeomorphic to its image under any embedding. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-topology
label:t-algebra$
51/28 Mathlib/Topology/Algebra/GroupWithZero.lean,Mathlib/Topology/Homeomorph/Lemmas.lean 2 1 ['github-actions'] nobody
20-28054
20 days ago
20-32309
20 days ago
20-32293
20 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 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
20-10483
20 days ago
20-18238
20 days ago
20-19618
20 days
24206 LessnessRandomness
author:LessnessRandomness
feat(Geometry/Euclidean/Angle/Unoriented): triangle inequality for angles Replace `proof_wanted` with proof. --- new-contributor t-euclidean-geometry awaiting-author 221/11 Mathlib.lean,Mathlib/Geometry/Euclidean/Angle/Unoriented/Affine.lean,Mathlib/Geometry/Euclidean/Angle/Unoriented/Basic.lean,Mathlib/Geometry/Euclidean/Angle/Unoriented/TriangleInequality.lean 4 16 ['LessnessRandomness', 'Timeroot', 'github-actions', 'jsm28', 'urkud'] jsm28
assignee:jsm28
19-77809
19 days ago
30-84002
30 days ago
20-6326
20 days
24928 kim-em
author:kim-em
chore: remove some `Nat` shortcut instances t-data 0/9 Mathlib/Algebra/Ring/Divisibility/Basic.lean,Mathlib/Data/List/TakeDrop.lean,Mathlib/Data/Nat/Basic.lean 3 10 ['Ruben-VandeVelde', 'github-actions', 'kim-em', 'leanprover-bot', 'leanprover-community-mathlib4-bot'] nobody
19-67618
19 days ago
19-67618
19 days ago
25-43867
25 days
25068 Parcly-Taxel
author:Parcly-Taxel
feat: IMO 2001 Q3 IMO 111/0 Archive.lean,Archive/Imo/Imo2001Q3.lean 2 1 ['github-actions'] nobody
19-64371
19 days ago
19-67128
19 days ago
19-67112
19 days
20240 mitchell-horner
author:mitchell-horner
feat(Combinatorics/SimpleGraph): prove the Kővári–Sós–Turán theorem Prove the Kővári–Sós–Turán theorem for simple graphs: the `(completeBipartiteGraph α β).Free` simple graphs for `card α ≤ card β` on the vertex type `V` have at most `(card β-1)^(1/(card α))*(card V)^(2-1/(card α))/2 + (card V)*(card α-1)/2` edges. --- - [x] depends on: #19865 - [x] depends on: #20738 I'd like to make `aux` not private in the `KovariSosTuran` namespace to enable reuse of the double-counting here, but I don't know what to call it. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-combinatorics 289/0 Mathlib.lean,Mathlib/Combinatorics/SimpleGraph/Bipartite.lean,Mathlib/Combinatorics/SimpleGraph/Extremal/KovariSosTuran.lean 3 3 ['github-actions', 'mathlib4-dependent-issues-bot'] awainverse
assignee:awainverse
19-29414
19 days ago
41-69299
1 month ago
41-69833
41 days
22018 maddycrim
author:maddycrim
feat(RingTheory/Localization/Pi): localization of a finite direct product where each semiring in product has maximal nilradical is a projection For noncomputable def `surjectivePiNilradicalIsMaximal` : Let `M` be a submonoid of a direct product of commutative rings `R i`. If each `R i` has maximal nilradical then the direct product `∏ R i` surjects onto the localization of `∏ R i` at `M`. --- [![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$
28/0 Mathlib/RingTheory/Localization/Pi.lean 1 24 ['Paul-Lez', 'alreadydone', 'erdOne', 'github-actions', 'grunweg', 'jcommelin', 'maddycrim'] mariainesdff
assignee:mariainesdff
19-29279
19 days ago
64-12686
2 months ago
110-85911
110 days
22961 xroblot
author:xroblot
feat(ZLattice/Covolume): add `covolume_div_covolume_eq_relindex` Add the following result: Let `L₁` be a sub-`ℤ`-lattice of `L₂`. Then the index of `L₁` inside `L₂` is equal to `covolume L₁ / covolume L₂`. --- - [x] depends on: #22940 - [x] depends on: #23759 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
66/4 Mathlib/Algebra/Module/ZLattice/Basic.lean,Mathlib/Algebra/Module/ZLattice/Covolume.lean,Mathlib/GroupTheory/Index.lean,Mathlib/LinearAlgebra/Determinant.lean 4 10 ['Ruben-VandeVelde', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'xroblot'] ericrbg
assignee:ericrbg
19-29255
19 days ago
42-41084
1 month ago
78-83644
78 days
23681 Timeroot
author:Timeroot
feat(Algebra/Polynomial): Descartes' Rule of signs Proof of Descartes' Rule of Signs. Last PR from https://github.com/Timeroot/lean-descartes-signs , now that #9085 is merged. Defines `Polynomial.SignVariations` as the relevant quantity, and `descartes_rule_of_signs` as the headline theorem. --- I tried to clean it up + golf it down and did shrink it a good deal. The lemma `signvar_mul_eraseLead_le_of_nextCoeff` is still 142 lines, and `succ_sign_lin_mul` is ~140 lines of code as well. Those are the ugly ones. I welcome ideas if someone wants to try to clean them up more! But the proof really does require an annoying bit of case-splitting, as far as I can tell. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
615/3 Mathlib.lean,Mathlib/Algebra/Polynomial/CoeffList.lean,Mathlib/Algebra/Polynomial/Degree/Operations.lean,Mathlib/Algebra/Polynomial/EraseLead.lean,Mathlib/Algebra/Polynomial/RuleOfSigns.lean 5 6 ['BoltonBailey', 'Timeroot', 'github-actions', 'grunweg'] adomani
assignee:adomani
19-28937
19 days ago
65-82525
2 months ago
65-82572
65 days
24260 plp127
author:plp127
feat(Topology): add API for Hereditarily Lindelof spaces Copies the stuff about Lindelof spaces to Hereditarily Lindelof spaces. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology awaiting-author 222/42 Mathlib/Topology/Compactness/Lindelof.lean 1 14 ['github-actions', 'grunweg', 'urkud'] urkud
assignee:urkud
19-28651
19 days ago
19-28690
19 days ago
29-42365
29 days
24931 qawbecrdtey
author:qawbecrdtey
feat(Data/Nat/Sqrt): Added lemma `Nat.add_one_sqrt_le_of_pos` --- This commit proves a single lemma `Nat.add_one_sqrt_le_of_pos`. ```lean lemma add_one_sqrt_le_of_pos {n : ℕ} (hn : 1 ≤ n) : (n + 1).sqrt ≤ n ``` [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data easy 7/0 Mathlib/Data/Nat/Sqrt.lean 1 4 ['Ruben-VandeVelde', 'eric-wieser', 'github-actions', 'qawbecrdtey'] nobody
19-23003
19 days ago
25-37853
25 days ago
25-37911
25 days
23752 jsm28
author:jsm28
feat(Geometry/Euclidean/Incenter): incenters and excenters Define the exspheres and insphere of a simplex (in dimension 1 and greater), and corresponding definitions for their center and radius. Give necessary and sufficient conditions for them to exist (in terms of the barycentric coordinates, being signed versions of the inverses of the distances between vertices and opposite faces, having a nonzero sum) and show that they do always exist in the case of the incenter and of the excenter opposite a single vertex (the latter in dimensions 2 and greater), and that any point lying in the span of the vertices and equidistant from the faces opposite the vertices is an excenter (and, when signs of the equal distances are given, is the excenter with corresponding signs). Some major pieces are deferred to followups, in particular definitions of touchpoints, tangency of exspheres and insphere to faces, and the relation to angle bisectors in various forms. But since the file is already over 600 lines, I think this is a reasonable starting point (and since the lemmas do show that the definitions have their characteristic properties of points being equidistant from the faces on the desired sides, I think it sufficiently justifies that the definitions are correct and usable as-is). Feel free to golf; the calculations involved in showing that the excenter opposite a vertex always exists (in dimensions 2 and greater) are rather long. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) - [x] depends on: #23712 - [x] depends on: #23751 - [x] depends on: #24503 - [x] depends on: #24968 - [x] depends on: #25029 t-euclidean-geometry 556/0 Mathlib.lean,Mathlib/Data/Fin/Basic.lean,Mathlib/Geometry/Euclidean/Altitude.lean,Mathlib/Geometry/Euclidean/Incenter.lean 4 53 ['JovanGerb', 'eric-wieser', 'github-actions', 'jsm28', 'mathlib4-dependent-issues-bot'] eric-wieser
assignee:eric-wieser
19-26
19 days ago
20-11713
20 days ago
62-48480
62 days
25096 CBirkbeck
author:CBirkbeck
feat(Analysis/NormedSpace/FunctionSeries): Add SummableUniformlyOn ve… …rsions and derivwithin_tsum --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-analysis 43/2 Mathlib/Analysis/NormedSpace/FunctionSeries.lean 1 1 ['github-actions'] nobody
18-80632
18 days ago
18-82404
18 days ago
0-0
0 seconds
24333 xcloudyunx
author:xcloudyunx
feat(Combinatorics/SimpleGraph): cycle graph implementation for generic vertex types The existing `cycleGraph` implementation under Combinatorics/SimpleGraph/Circulant.lean only operates over `Fin n`. This PR implements a cycle graph implementation over any generic vertex type. --- [![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
18-68272
18 days ago
46-65829
1 month ago
46-65883
46 days
24703 robin-carlier
author:robin-carlier
feat(CategoryTheory/Monoidal): external product of diagrams in monoidal categories Given functors `K₁ : J₁ ⥤ C` and `K₂ : J₂ ⥤ C` with values in a monoidal category, define a construction `externalProduct K₁ K₂` (denoted `K₁ ⊠ K₂`) as the bifunctor `(j₁, j₂) ↦ K₁ j₁ ⊗ K₂ j₂`. We show that composition of this construction with the diagonal functor to the product recovers the pointwise tensor product of functors, and we show that this construction satisfies a symmetry whenever `C` is braided. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory 99/0 Mathlib.lean,Mathlib/CategoryTheory/Monoidal/ExternalProduct.lean 2 5 ['github-actions', 'joelriou'] nobody
18-47098
18 days ago
18-47161
18 days ago
31-2826
31 days
21673 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/) t-analysis 329/0 Mathlib.lean,Mathlib/Algebra/BigOperators/Group/Finset/Disjoint.lean,Mathlib/Algebra/Module/ZLattice/Summable.lean,Mathlib/Order/Disjointed.lean 4 4 ['github-actions', 'leanprover-community-bot-assistant', 'xroblot'] nobody
18-39201
18 days ago
18-39224
18 days ago
46-26084
46 days
16074 Rida-Hamadani
author:Rida-Hamadani
feat: combinatorial maps and planar graphs We define combinatorial maps, then we define planar graph using combinatorial maps. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics 243/0 Mathlib.lean,Mathlib/Combinatorics/SimpleGraph/Planar.lean,Mathlib/Data/CombinatorialMap.lean 3 27 ['Parcly-Taxel', 'Rida-Hamadani', 'github-actions', 'lambda-fairy', 'leanprover-community-bot-assistant'] kmill
assignee:kmill
18-24212
18 days ago
43-35814
1 month ago
47-23245
47 days
21838 joneugster
author:joneugster
feat(Cache): Allow arguments of the form `Mathlib.Data` which correspond to a folder but not a file --- - [x] depends on: #21834 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) CI t-meta awaiting-author 34/11 Cache/IO.lean,Cache/Main.lean 2 10 ['eric-wieser', 'github-actions', 'joneugster', 'mathlib4-dependent-issues-bot', 'mergify'] nobody
18-24127
18 days ago
18-24127
18 days ago
50-67617
50 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
18-24063
18 days ago
54-35449
1 month ago
109-82571
109 days
23926 b-reinke
author:b-reinke
feat(Algebra/BigOperators/Finprod): add powerset projection lemmas This PR adds lemmas in `Mathlib/Algebra/BigOperators/Finprod.lean` related to products/sums over the powerset `𝒫 s` when we add or remove an element of `s`. The motivation comes from the proof of the deletion/contraction properties of matroids. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
30/0 Mathlib/Algebra/BigOperators/Finprod.lean,Mathlib/Data/Set/Image.lean 2 5 ['b-reinke', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant'] joelriou
assignee:joelriou
18-23928
18 days ago
46-44557
1 month ago
59-45080
59 days
24139 yuanyi-350
author:yuanyi-350
feat: add `Fin.cycleIcc` which rotates `range(i, j)` In this file, I define permutation `cycleIcc i j hij`, which is the cycle `(i i+1 .... j)` leaving `(0 ... i-1)` and `(j+1 ... n-1)` unchanged. In other words, it rotates elements in `[i, j]` one step to the right. Also I prove some properties of `cycleIcc i j hij` such as it is a cycle and its cycleType is `j - i` **This definition is used to prove the following result:** ``` theorem succAbove_comp_cycleIcc [NeZero n] (x : Fin (n + 1) → L) (i j : Fin (n + 1)) (eq : x i = x j) (lt : i < j) x ∘ i.succAbove = x ∘ j.succAbove ∘ (cycleIcc hij) ``` More clearly, `x ∘ i.succAbove` and `x ∘ j.succAbove` are `Fin n → L` types. For example, when `n = 6, i = 2, j = 5` and `x i = x j` ``` x ∘ i.succAbove = (x 0, x 1, x 3, x 4, x 5, x 6) x ∘ j.succAbove = (x 0, x 1, x 2, x 3, x 4, x 6) ``` We have ``` (x 0, x 1, x 3, x 4, x 5, x 6) --(cycleIcc)--->(x 0, x 1, x 5, x 3, x 4, x 6) = (x 0, x 1, x 2, x 3, x 4, x 6) ``` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra
label:t-algebra$
132/1 Mathlib/Algebra/Group/Fin/Basic.lean,Mathlib/Data/Fin/Basic.lean,Mathlib/Data/Nat/SuccPred.lean,Mathlib/GroupTheory/Perm/Fin.lean 4 27 ['acmepjz', 'faenuccio', 'github-actions', 'grunweg', 'leanprover-bot', 'leanprover-community-bot-assistant', 'mbkybky', 'yuanyi-350'] faenuccio
assignee:faenuccio
18-23587
18 days ago
38-69996
1 month ago
52-84299
52 days
24546 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/) t-combinatorics 36/0 Mathlib/Combinatorics/SimpleGraph/Coloring.lean,Mathlib/Combinatorics/SimpleGraph/ConcreteColorings.lean,Mathlib/Combinatorics/SimpleGraph/Path.lean 3 3 ['IvanRenison', 'github-actions', 'jt496'] b-mehta
assignee:b-mehta
18-23441
18 days ago
38-24851
1 month ago
38-40361
38 days
21966 vasnesterov
author:vasnesterov
feat(Tactic/Order): support `⊤`, `⊥`, and lattice operations Support `⊤`, `⊥`, and lattice operations in the `order` tactic. --- - [x] depends on: #21877 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-meta 255/81 Mathlib/Tactic/Order.lean,Mathlib/Tactic/Order/CollectFacts.lean,Mathlib/Tactic/Order/Graph/Basic.lean,Mathlib/Tactic/Order/Preprocessing.lean,MathlibTest/order.lean,scripts/noshake.json 6 2 ['github-actions', 'mathlib4-dependent-issues-bot'] kmill
assignee:kmill
18-21038
18 days ago
67-38583
2 months ago
101-35078
101 days
22100 smmercuri
author:smmercuri
feat: two inequivalent absolute values have a `< 1` and `> 1` value - Two absolute values `v` and `w` are equivalent if and only if `v x < 1` exactly when `w x < 1` - Two inequivalent absolute values `v` and `w` have a point `x` at which `1 < v x` and `w x < 1` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-analysis awaiting-author
label:t-algebra$
176/0 Mathlib/Algebra/Order/AbsoluteValue/Basic.lean,Mathlib/Analysis/AbsoluteValue/Equivalence.lean 2 13 ['Paul-Lez', 'faenuccio', 'github-actions', 'smmercuri'] faenuccio
assignee:faenuccio
18-13427
18 days ago
18-13427
18 days ago
65-54803
65 days
25101 erdOne
author:erdOne
feat(AlgebraicGeometry): building morphisms into Proj --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebraic-geometry 231/3 Mathlib/AlgebraicGeometry/ProjectiveSpectrum/Basic.lean,Mathlib/AlgebraicGeometry/Restrict.lean,Mathlib/AlgebraicGeometry/Scheme.lean,Mathlib/RingTheory/GradedAlgebra/HomogeneousLocalization.lean 4 6 ['erdOne', 'github-actions', 'joelriou'] nobody
17-78571
17 days ago
17-78571
17 days ago
18-58260
18 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'] nobody
17-68079
17 days ago
17-68079
17 days ago
17-68132
17 days
25124 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 1 ['github-actions'] nobody
17-63123
17 days ago
17-65948
17 days ago
17-65991
17 days
24485 dagurtomas
author:dagurtomas
feat(CategoryTheory): localization preserves braided structure --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory 733/427 Mathlib.lean,Mathlib/CategoryTheory/Localization/Monoidal.lean,Mathlib/CategoryTheory/Localization/Monoidal/Basic.lean,Mathlib/CategoryTheory/Localization/Monoidal/Braided.lean,Mathlib/CategoryTheory/Monoidal/Braided/Basic.lean,Mathlib/CategoryTheory/Sites/Monoidal.lean 6 7 ['dagurtomas', 'github-actions', 'joelriou', 'leanprover-community-bot-assistant'] nobody
17-41565
17 days ago
17-41565
17 days ago
27-82564
27 days
24651 Hagb
author:Hagb
feat(RingTheory/Finiteness/Defs): span of a set is finitely generated iff generated by a finite subset --- - [ ] depends on: #24648 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra
label:t-algebra$
14/0 Mathlib/RingTheory/Finiteness/Defs.lean 1 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
17-38635
17 days ago
17-38654
17 days ago
17-43206
17 days
23365 vasnesterov
author:vasnesterov
feat(Tactic/Simproc): nested quantifiers in `existsAndEq` Generalize the `existsAndEq` simproc to nested existential quantifiers. For example `∃ a, p a ∧ ∃ b, a = f b ∧ q b` now simplifies to `∃ b, p (f b) ∧ q b`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-meta 440/73 Mathlib/Tactic/Simproc/ExistsAndEq.lean,MathlibTest/Simproc/ExistsAndEq.lean 2 41 ['JovanGerb', 'b-mehta', 'eric-wieser', 'github-actions', 'grunweg', 'kim-em', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'vasnesterov'] nobody
17-36555
17 days ago
67-74040
2 months ago
73-14281
73 days
24350 erdOne
author:erdOne
feat(FieldTheory): fg extension over perfect field is separably generated Co-authored-by: Christian Merten --- - [x] depends on: #24344 - [x] depends on: #24346 - [x] depends on: #24347 - [x] depends on: #24348 - [x] depends on: #24349 - [ ] depends on: #25062 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra blocked-by-other-PR WIP
label:t-algebra$
465/0 Mathlib.lean,Mathlib/FieldTheory/SeparablyGenerated.lean 2 3 ['erdOne', 'github-actions', 'mathlib4-dependent-issues-bot'] nobody
17-35016
17 days ago
17-35017
17 days ago
0-16
16 seconds
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'] nobody
17-25545
17 days ago
17-25612
17 days ago
34-10636
34 days
22931 chrisflav
author:chrisflav
refactor(RingTheory/RingHom): factor out proofs for `Algebra.FiniteType` 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.FiniteType` 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: #22933 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
126/119 Mathlib/RingTheory/FiniteType.lean,Mathlib/RingTheory/RingHom/Finite.lean,Mathlib/RingTheory/RingHom/FiniteType.lean 3 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
17-23901
17 days ago
17-25275
17 days ago
17-26487
17 days
25112 linesthatinterlace
author:linesthatinterlace
feat(`Algebra/Group/Prod`): Add API for inclusion and projection maps from and to the product of units. Adds API for inclusion and projection maps from and to the product of units. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
99/30 Mathlib/Algebra/BigOperators/Associated.lean,Mathlib/Algebra/Group/Prod.lean,Mathlib/Data/Nat/Totient.lean,Mathlib/Topology/Algebra/Group/Basic.lean 4 9 ['eric-wieser', 'github-actions', 'linesthatinterlace', 'pechersky'] nobody
17-23021
17 days ago
18-25288
18 days ago
18-25451
18 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'] nobody
17-16885
17 days ago
19-63787
19 days ago
19-63844
19 days
25135 vasnesterov
author:vasnesterov
WIP/test PR for faster `tauto` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-meta WIP 14/6 Mathlib/Geometry/Manifold/IsManifold/InteriorBoundary.lean,Mathlib/Tactic/Tauto.lean,scripts/noshake.json 3 4 ['github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot'] nobody
16-81351
16 days ago
16-81351
16 days ago
0-1
1 second
25133 erdOne
author:erdOne
feat(Tactic/NormNum): support positive characteristic Co-authored-by: Heather Macbeth --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-meta WIP 250/39 Mathlib/Tactic/NormNum/CharP.lean,Mathlib/Tactic/NormNum/Core.lean,Mathlib/Tactic/NormNum/Eq.lean,Mathlib/Tactic/NormNum/Inv.lean,Mathlib/Tactic/NormNum/Test.lean 5 4 ['erdOne', 'eric-wieser', 'github-actions'] nobody
16-74942
16 days ago
17-19962
17 days ago
0-0
0 seconds
11155 smorel394
author:smorel394
feat(LinearAlgebra/Multilinear/DirectSum, LinearAlgebra/DirectSum/{PiTensorProduct,Finsupp}): interaction between `MultilinearMap` and `DirectSum`, and between `PiTensorProduct` and `DirectSum` This does three things: * `MultilinearMap.fromDirectSumEquiv` (in `LinearAlgebra/MultilinearMap/DirectSum.lean`) calculates `MultilinearMap`s on a family of `DirectSum`s. More precisely, if `ι` is a `Fintype`, if `κ i` is a family of types indexed by `ι` and we have a `R`-module `M i j` for every `i : ι` and `j : κ i`, this is the linear equivalence between `Π p : (i : ι) → κ i, MultilinearMap R (fun i ↦ M i (p i)) M'` and `MultilinearMap R (fun i ↦ ⨁ j : κ i, M i j) M'`. * `PiTensorProduct.directSum` (in `LinearAlgebra/DirectSum/PiTensorProduct.lean`): the distributivity property of a `PiTensorProduct` with respect to `DirectSum`s in all its arguments. * `finsuppPiTensorProduct` (in `LinearAlgebra/DirectSum/Finsupp.lean`): If `ι` is a `Fintype`, `κ i` is a family of types indexed by `ι` and `M i` is a family of `R`-modules indexed by `ι`, then the tensor product of the family `κ i →₀ M i` is linearly equivalent to `∏ i, κ i →₀ ⨂[R] i, M i`. - [x] depends on: #11152 - [x] depends on: #11196 - [x] depends on: #17881 - [x] depends on: #17932 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra please-adopt
label:t-algebra$
322/0 Mathlib.lean,Mathlib/LinearAlgebra/DFinsupp/PiTensorProduct.lean,Mathlib/LinearAlgebra/DirectSum/Finsupp.lean,Mathlib/LinearAlgebra/DirectSum/PiTensorProduct.lean,Mathlib/LinearAlgebra/Multilinear/DFinsupp.lean,Mathlib/LinearAlgebra/Multilinear/DirectSum.lean 6 32 ['Ruben-VandeVelde', 'eric-wieser', 'github-actions', 'mathlib4-dependent-issues-bot', 'smorel394'] nobody
16-69178
16 days ago
16-71383
16 days ago
6-23591
6 days
25071 erdOne
author:erdOne
feat(EllipticCurve): basic API for singular cubics --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebraic-geometry 320/0 Mathlib.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Singular/Basic.lean,Mathlib/AlgebraicGeometry/EllipticCurve/VariableChange.lean 3 34 ['Multramate', 'acmepjz', 'erdOne', 'github-actions'] nobody
16-60121
16 days ago
19-61944
19 days ago
19-62000
19 days
23312 xroblot
author:xroblot
feat(NumberField/Units): prove that a family of units is of max rank iff its closure has finite index Let `u : Fin (rank K) → (𝓞 K)ˣ` be a family of units of a number field `K`. We prove that `isMaxRank u`, that is its regulator is nonzero, iff `closure (Set.range u))` has finite index. --- - [x] depends on: #22882 - [x] depends on: #23063 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-number-theory 70/3 Mathlib/GroupTheory/Index.lean,Mathlib/LinearAlgebra/FreeModule/Finite/Quotient.lean,Mathlib/NumberTheory/NumberField/Units/Regulator.lean 3 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
16-25473
16 days ago
16-25491
16 days ago
16-26436
16 days
25150 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/) t-category-theory 191/0 Mathlib.lean,Mathlib/CategoryTheory/Bicategory/LocallyGroupoid.lean 2 1 ['github-actions'] nobody
16-15580
16 days ago
16-19133
16 days ago
16-19188
16 days
24497 Parcly-Taxel
author:Parcly-Taxel
feat: IMO 1985 Q2 IMO 100/0 Archive.lean,Archive/Imo/Imo1985Q2.lean 2 1 ['github-actions'] dwrensha
assignee:dwrensha
16-10479
16 days ago
39-37793
1 month ago
39-37776
39 days
24517 upobir
author:upobir
feat(Algebra/QuadraticDiscriminant): Adding inequalities on quadratic from inequalities on discriminant --- This pr adds inequalities that relate `0` and `a * (x * x) + b * x + c` from inequalities of `a` and `discrim a b c`. For example, negative discriminant and negative leading coefficient implies value of quadratic expression is always negative and similar. [![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 1 ['github-actions'] chrisflav
assignee:chrisflav
16-10458
16 days ago
39-16657
1 month ago
39-16709
39 days
24522 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/) t-condensed 39/0 Mathlib.lean,Mathlib/Condensed/Light/Small.lean 2 1 ['github-actions'] joneugster
assignee:joneugster
16-10408
16 days ago
39-9950
1 month ago
39-10005
39 days
24685 robin-carlier
author:robin-carlier
feat(CategoryTheory/Limits/Preserves): Preservations of (co)limits by bifunctors Introduce a typeclass `PreservesColimit₂` that bundles the assumption that a bifunctor preserves a pair of colimit diagrams in each of its variables. This is stated in terms of a construction `Functor.mapCocone₂` that applies a bifunctor `G` to a pair of cocones to get a cocone over the uncurryfication of `whiskeringLeft₂ _|>.obj _|>.obj _|>.obj G`. The cocone points of this construction is definitionally the evaluation of `G` at the cocone points of the two cocones given as parameters. We give helper functions to extract isomorphisms with abstract colimits out of this typeclass, and we characterize these isomorphisms with respect to the canonical maps to the colimits. The dual typeclass for limits is also introduced. --- The definition of `Functor.mapCocone₂` and of `PreservesColimit₂` is due to @joelriou and was suggested during review of #17781. This PR only contains basic definitions, but does not give any interesting ways of inferring a `PreservesColimit₂` instance. This will be the content of a follow-up PR. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory 243/0 Mathlib.lean,Mathlib/CategoryTheory/Limits/Preserves/Bifunctor.lean 2 1 ['github-actions'] joelriou
assignee:joelriou
16-10290
16 days ago
32-15906
1 month ago
32-15960
32 days
19456 AntoineChambert-Loir
author:AntoineChambert-Loir
feat(Data/Finsupp/MonomialOrder/DegRevLex): homogeneous reverse lexicographic order Definition of the homogeneous reverse lexicographic order --- - [x] depends on: #19453 - [x] depends on: #19455 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data t-order t-algebraic-geometry WIP 362/0 Mathlib.lean,Mathlib/Data/Finsupp/MonomialOrder/DegLex.lean,Mathlib/Data/Finsupp/MonomialOrder/DegRevLex.lean 3 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
16-8835
16 days ago
16-8835
16 days ago
0-1720
28 minutes
24213 BoltonBailey
author:BoltonBailey
feat: add simp lemmas for trig functions on `π * 2⁻¹` This PR adds a number of simp lemmas to reduce trig functions evaluated on `π * 2⁻¹`. This allows `simp` to reduce expressions such as `sin (π * (1 / 2))` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis 45/0 Mathlib/Analysis/SpecialFunctions/Trigonometric/Basic.lean 1 3 ['YaelDillies', 'github-actions', 'leanprover-community-bot-assistant'] YaelDillies
assignee:YaelDillies
16-2360
16 days ago
31-9258
1 month ago
49-66650
49 days
21103 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`. --- - [x] depends on: #21098 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory 118/5 Mathlib/AlgebraicTopology/SimplexCategory/Basic.lean,Mathlib/AlgebraicTopology/SimplicialSet/Degenerate.lean 2 5 ['dagurtomas', 'gio256', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
15-86359
15 days ago
51-83505
1 month ago
90-28708
90 days
5863 eric-wieser
author:eric-wieser
feat: add elaborators for concrete matrices --- - [x] depends on: #5866 - [ ] depends on: #5897 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta blocked-by-other-PR help-wanted 257/7 Mathlib/Control/Monad/Cont.lean,Mathlib/Data/Matrix/Auto.lean,MathlibTest/matrix_auto.lean 3 7 ['eric-wieser', 'github-actions', 'kim-em', 'leanprover-community-bot-assistant'] nobody
15-79369
15 days ago
15-79390
15 days ago
0-0
0 seconds
25157 wwylele
author:wwylele
feat(Data/Real): add embedding of archimedean groups into Real This is part of #25140, and is the special case of Hahn embedding theorem applied to archimedean group. The construction is rather unpleasant as it uses explicit Cauchy sequence with essentially the binary representation of numbers, but I haven't found a better way to do this. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data 288/0 Mathlib.lean,Mathlib/Data/Real/Embedding.lean 2 3 ['eric-wieser', 'github-actions', 'wwylele'] nobody
15-74090
15 days ago
16-11777
16 days ago
16-11830
16 days
25105 erdOne
author:erdOne
feat(AlgebraicGeometry): inverse limit of nonempty quasicompact closeds is nonempty --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-algebraic-geometry 92/2 Mathlib/AlgebraicGeometry/AffineTransitionLimit.lean,Mathlib/AlgebraicGeometry/Morphisms/Separated.lean,Mathlib/CategoryTheory/Comma/Over/Basic.lean 3 1 ['github-actions'] nobody
15-64061
15 days ago
18-42130
18 days ago
18-42182
18 days
23547 chrisflav
author:chrisflav
feat(AlgebraicGeometry): codescent implies descent Let `P` and `P'` be morphism properties of schemes. We show some results to deduce that `P` descends along `P'` from a codescent property of ring homomorphisms. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebraic-geometry awaiting-author 258/1 Mathlib.lean,Mathlib/AlgebraicGeometry/Morphisms/AffineAnd.lean,Mathlib/AlgebraicGeometry/Morphisms/Descent.lean,Mathlib/RingTheory/RingHomProperties.lean 4 15 ['chrisflav', 'erdOne', 'github-actions'] erdOne
assignee:erdOne
15-63881
15 days ago
15-63881
15 days ago
50-4378
50 days
24816 ciskiko
author:ciskiko
feat(GroupTheory): add Regular Wreath Product feat: add regular wreath product and some results; add iterated wreath product; add the isomorphism of iterated wreath product of Z_p to sylow p subgroup of S_{p^n}. Needs some work simplifying final result. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) maintainer-merge new-contributor t-algebra
label:t-algebra$
285/1 Mathlib.lean,Mathlib/Algebra/Group/End.lean,Mathlib/Combinatorics/Additive/AP/Three/Behrend.lean,Mathlib/Data/Nat/Multiplicity.lean,Mathlib/GroupTheory/RegularWreathProduct.lean,Mathlib/Logic/Equiv/Fin/Basic.lean,Mathlib/SetTheory/Cardinal/Finite.lean 7 102 ['ciskiko', 'github-actions', 'tb65536'] tb65536
assignee:tb65536
15-33430
15 days ago
15-33431
15 days ago
24-38027
24 days
24819 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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
27/3 Mathlib/RingTheory/MvPolynomial/Groebner.lean 1 4 ['Hagb', 'github-actions'] nobody
15-12814
15 days ago
28-6092
28 days ago
28-6144
28 days
21283 erdOne
author:erdOne
feat: topology on Hom(R, S) in `CommRingCat` Co-authored-by: Christian Merten --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-topology
label:t-algebra$
239/0 Mathlib.lean,Mathlib/Algebra/Category/Ring/Constructions.lean,Mathlib/Algebra/Category/Ring/Topology.lean,Mathlib/RingTheory/TensorProduct/Basic.lean,Mathlib/Topology/Constructions.lean,Mathlib/Topology/Homeomorph/Lemmas.lean,scripts/noshake.json 7 21 ['dagurtomas', 'erdOne', 'github-actions', 'kbuzzard'] nobody
15-7653
15 days ago
27-12564
27 days ago
109-40479
109 days
24103 plp127
author:plp127
feat(Topology/UniformSpace/OfCompactT2): generalize theorem Generalize `uniformSpaceOfCompactT2` to `uniformSpaceOfCompactR1`. --- - [ ] depends on: #24098 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology 48/24 Mathlib/Topology/Separation/Regular.lean,Mathlib/Topology/UniformSpace/OfCompactT2.lean 2 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
15-3140
15 days ago
15-3162
15 days ago
46-79521
46 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 14 ['YaelDillies', 'erdOne', 'eric-wieser', 'github-actions'] nobody
15-2432
15 days ago
15-2493
15 days ago
15-6417
15 days
25197 eric-wieser
author:eric-wieser
feat: Finset.sum induction for tensor products. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-algebra
label:t-algebra$
81/0 Mathlib/LinearAlgebra/TensorProduct/Basic.lean 1 1 ['github-actions'] nobody
14-72847
14 days ago
14-72854
14 days ago
0-0
0 seconds
23368 b-reinke
author:b-reinke
feat(GroupTheory/FreeGroup/ReducedWords): add theory of reduced words Upstreamed from the [EquationalTheories](https://github.com/teorth/equational_theories) project. This PR adds the file `GroupTheory/FreeGroup/ReducedWords.lean`, where the predicate of reduced words is defined. It is shown that `reduce` and `toWord` produce reduced words. This is done in preparation for the theory of cyclically reduced words. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-geometric-group-theory t-algebra
label:t-algebra$
104/0 Mathlib.lean,Mathlib/GroupTheory/FreeGroup/ReducedWords.lean 2 37 ['b-reinke', 'github-actions', 'tb65536', 'vlad902'] nobody
14-59970
14 days ago
74-25781
2 months ago
74-33611
74 days
25188 vlad902
author:vlad902
feat: add lemmas about `List.scanr` I add basic lemmas to reason about `List.scanr`, and slightly clean-up the file and add some basic lemmas to keep the API unified with the one for `List.scanl`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data 84/18 Mathlib/Data/List/Scan.lean 1 5 ['b-mehta', 'github-actions', 'vlad902'] nobody
14-48841
14 days ago
14-49069
14 days ago
14-72569
14 days
25204 YaelDillies
author:YaelDillies
refactor: redefine `ProperCone` as an `abbrev` for `ClosedSubmodule` ... and derive the `ProperCone` operations from `ClosedSubmodule` too. Also rename the scalar ring from `𝕜` to `R`. From Toric --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) toric t-analysis 79/90 Mathlib/Analysis/Convex/Cone/Proper.lean 1 1 ['github-actions'] nobody
14-37093
14 days ago
14-37135
14 days ago
14-37146
14 days
24862 grunweg
author:grunweg
feat(LocallyIntegrable): generalise more to enorms --- - [ ] depends on: #24352 - [ ] open question: filter lemmas; IsBoundedUnder is not the right condition as-is; need to think (or just not generalise) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) carleson t-measure-probability WIP 171/88 Mathlib/MeasureTheory/Function/L1Space/HasFiniteIntegral.lean,Mathlib/MeasureTheory/Function/LocallyIntegrable.lean,Mathlib/MeasureTheory/Integral/IntegrableOn.lean 3 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
14-30975
14 days ago
14-30975
14 days ago
0-1
1 second
8102 miguelmarco
author:miguelmarco
feat(Tactic): add `unify_denoms` and `collect_signs` tactics This PR adds four new tactics: - `unify_denoms` tries to put expressions with several divisions in a form with only one division. In the case of fields, it works similarly to `field_simp`, but if the hypothesis about denominators being nonzero are not present, it assumes them, and leaves them as new goals to prove. In that sense, it is an "unsafe" tactic (but can be useful nevertheless, for example when you can't find which exact hypothesis is missing). It also works with expressions of naturals and Euclidean domains, assuming the corresponding hypothesis about the denominators dividing the numerators. - `unify_denoms!` extends `unify_denoms` to work with (in)equalities, assuming also that the denominators, once in normal form, are positive. - `collect_signs` works similarly with expressions using sums and substractions: it tries to put them in a form of one sum minus other sum. In the case of working with naturals, it assumes that we never substract a bigger number from a smaller one. Both are implemented essentially as a macro that combines several rewriting rules. Some new lemmas with the corresponding rules are added. --- new-contributor t-meta please-adopt modifies-tactic-syntax good first issue 407/0 Mathlib.lean,Mathlib/Algebra/EuclideanDomain/Basic.lean,Mathlib/Tactic.lean,Mathlib/Tactic/CollectSigns.lean,Mathlib/Tactic/UnifyDenoms.lean,MathlibTest/unify_denoms.lean,scripts/noshake.json 7 54 ['Paul-Lez', 'YaelDillies', 'github-actions', 'joneugster', 'kbuzzard', 'miguelmarco'] Paul-Lez
assignee:Paul-Lez
14-24186
14 days ago
26-4939
26 days ago
22-16933
22 days
25209 upobir
author:upobir
feat(NumberTheory/Divisors): add int divisors --- this PR adds `Int.divisors` analogous to `Nat.divisors`. Some preliminary results are proven for the new definition. Imports have also been modified by using `#min_imports` [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-number-theory 125/4 Mathlib/NumberTheory/Divisors.lean 1 8 ['Paul-Lez', 'eric-wieser', 'github-actions', 'upobir'] nobody
14-18151
14 days ago
14-24775
14 days ago
14-24832
14 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
14-10564
14 days ago
55-85262
1 month ago
55-85314
55 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
14-1019
14 days ago
19-63820
19 days ago
19-63817
19 days
24753 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 --- - [ ] depends on: #21966 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-meta blocked-by-other-PR 578/59 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Order.lean,Mathlib/Tactic/Order/CollectFacts.lean,Mathlib/Tactic/Order/Graph/Basic.lean,Mathlib/Tactic/Order/Preprocessing.lean,Mathlib/Tactic/Order/ToInt.lean,MathlibTest/order.lean,scripts/noshake.json 9 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'plp127'] nobody
14-30
14 days ago
29-27982
29 days ago
0-654
10 minutes
25208 erdOne
author:erdOne
feat(LinearAlgebra): `tensor_induction` macro --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra RFC WIP
label:t-algebra$
87/116 Mathlib/Algebra/Category/ModuleCat/ChangeOfRings.lean,Mathlib/Algebra/Central/TensorProduct.lean,Mathlib/LinearAlgebra/DirectSum/Finsupp.lean,Mathlib/LinearAlgebra/TensorProduct/Basic.lean,Mathlib/RingTheory/Flat/Equalizer.lean,Mathlib/RingTheory/TensorProduct/Basic.lean,Mathlib/RingTheory/TensorProduct/Finite.lean,Mathlib/RingTheory/Unramified/Finite.lean 8 7 ['chrisflav', 'eric-wieser', 'github-actions', 'leanprover-bot'] nobody
13-84587
13 days ago
14-26594
14 days ago
0-600
10 minutes
23848 emilyriehl
author:emilyriehl
feat(AlgebraicTopology/SimplicialSet/NerveAdjunction): to Strict Segal 2 Under a suitable hypothesis, a map of 2-truncated simplicial sets can be generated from a refl prefunctor between the underlying reflexive quivers --- provided the codomain is `StrictSegal`. This abstracts a previously formalized result that requires the codomain to be the 2-truncated nerve of a category. Co-authored-by: Aaron Liu --- The current draft displays the old code for comparison with new versions labeled ALT. After initial review this will be cut. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) infinity-cosmos t-topology t-category-theory 490/202 Mathlib/AlgebraicTopology/SimplexCategory/Basic.lean,Mathlib/AlgebraicTopology/SimplicialSet/HomotopyCat.lean,Mathlib/AlgebraicTopology/SimplicialSet/NerveAdjunction.lean,Mathlib/AlgebraicTopology/SimplicialSet/StrictSegal.lean,Mathlib/CategoryTheory/ComposableArrows.lean,Mathlib/CategoryTheory/EqToHom.lean 6 17 ['emilyriehl', 'github-actions', 'joelriou'] nobody
13-65658
13 days ago
20-7827
20 days ago
26-75823
26 days
25182 YaelDillies
author:YaelDillies
feat: `(M →* N₁) ≃* (M →* N₂)` if `N₁ ≃* N₂` From Toric --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) toric t-algebra
label:t-algebra$
63/12 Mathlib/Algebra/Category/Grp/ForgetCorepresentable.lean,Mathlib/Algebra/Category/Grp/LargeColimits.lean,Mathlib/Algebra/Category/MonCat/ForgetCorepresentable.lean,Mathlib/Algebra/Group/Equiv/Basic.lean,Mathlib/GroupTheory/FiniteAbelian/Duality.lean 5 10 ['YaelDillies', 'eric-wieser', 'github-actions'] nobody
13-48712
13 days ago
14-41952
14 days ago
15-32593
15 days
21745 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/) large-import t-topology t-category-theory 253/7 Mathlib/AlgebraicTopology/SimplexCategory/GeneratorsRelations/NormalForms.lean 1 21 ['dagurtomas', 'github-actions', 'joelriou', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'robin-carlier'] nobody
13-47257
13 days ago
25-41685
25 days ago
48-49632
48 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 3 ['github-actions', 'leanprover-community-bot-assistant'] ericrbg
assignee:ericrbg
13-26690
13 days ago
13-26707
13 days ago
91-48456
91 days
23979 AntoineChambert-Loir
author:AntoineChambert-Loir
feat: Multiple Primitivity of group actions An action of a group G on a type X is n-primitive if it is n-transitive and if, for every subset s of cardinality n of X, the action of `fixingSubgroup G s` on the complement of `s` is primitive. This PR develops the basics of this notion. --- - [ ] depends on: #23970 - [x] depends on: #23962 - [x] depends on: #24107 - [x] depends on: #24167 - [x] depends on: #24117 - [x] depends on: #23386 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra blocked-by-other-PR
label:t-algebra$
796/5 Mathlib.lean,Mathlib/Algebra/Group/End.lean,Mathlib/GroupTheory/GroupAction/FixingSubgroup.lean,Mathlib/GroupTheory/GroupAction/MultiplePrimitivity.lean,Mathlib/GroupTheory/GroupAction/MultipleTransitivity.lean,Mathlib/GroupTheory/GroupAction/Primitive.lean,Mathlib/GroupTheory/GroupAction/SubMulAction.lean,Mathlib/GroupTheory/GroupAction/SubMulAction/OfFixingSubgroup.lean 8 9 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] riccardobrasca
assignee:riccardobrasca
13-20190
13 days ago
13-30604
13 days ago
0-12
12 seconds
25240 IvanRenison
author:IvanRenison
feat(Analysis/InnerProductSpace/Projection): add lemma `Submodule.le_iff_orthogonal_le_orthogonal` and similars --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis 25/0 Mathlib/Analysis/InnerProductSpace/Projection.lean 1 1 ['github-actions'] nobody
13-15930
13 days ago
13-15933
13 days ago
13-15986
13 days
23684 alreadydone
author:alreadydone
feat(RingTheory): integral extensions of comm. rings are local homs --- The import increase only affects one file so I hope it's okay. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-algebra
label:t-algebra$
57/65 Mathlib/Algebra/Field/Equiv.lean,Mathlib/Algebra/Group/Invertible/Basic.lean,Mathlib/Algebra/GroupWithZero/Units/Basic.lean,Mathlib/AlgebraicGeometry/Morphisms/Proper.lean,Mathlib/FieldTheory/LinearDisjoint.lean,Mathlib/LinearAlgebra/Dimension/Localization.lean,Mathlib/RingTheory/Artinian/Ring.lean,Mathlib/RingTheory/IntegralClosure/Algebra/Defs.lean,Mathlib/RingTheory/IntegralClosure/IsIntegralClosure/Basic.lean,Mathlib/RingTheory/LinearDisjoint.lean,Mathlib/RingTheory/Localization/FractionRing.lean,Mathlib/RingTheory/Localization/Integral.lean,Mathlib/RingTheory/SimpleRing/Field.lean 13 4 ['alreadydone', 'github-actions', 'xroblot'] nobody
13-6805
13 days ago
65-72197
2 months ago
65-72217
65 days
25224 xcloudyunx
author:xcloudyunx
feat(Combinatorics/SimpleGraph): edgeSet of Eulerian walk equal to edgeSet of graph --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-combinatorics easy 6/0 Mathlib/Combinatorics/SimpleGraph/Trails.lean 1 2 ['IvanRenison', 'github-actions'] nobody
12-83709
12 days ago
13-74712
13 days ago
13-75614
13 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'] nobody
12-83102
12 days ago
13-74514
13 days ago
13-74571
13 days
24120 AntoineChambert-Loir
author:AntoineChambert-Loir
feat(GroupTheory/GroupAction/Jordan) : Primitivity lemmas This is a primitivity lemma for actions, in preparation to the proof of of Jordan on primitive subgroups of the permutation group #24131. --- - [x] depends on: #24167 - [x] depends on: #24117 - [x] depends on: #24107 - [x] depends on: #23962 - [x] depends on: #23386 - [ ] depends on: #23979 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra blocked-by-other-PR
label:t-algebra$
1573/6 Mathlib.lean,Mathlib/Algebra/Group/End.lean,Mathlib/GroupTheory/GroupAction/FixingSubgroup.lean,Mathlib/GroupTheory/GroupAction/Jordan.lean,Mathlib/GroupTheory/GroupAction/MultiplePrimitivity.lean,Mathlib/GroupTheory/GroupAction/MultipleTransitivity.lean,Mathlib/GroupTheory/GroupAction/Primitive.lean,Mathlib/GroupTheory/GroupAction/SubMulAction.lean,Mathlib/GroupTheory/GroupAction/SubMulAction/OfFixingSubgroup.lean 9 7 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] riccardobrasca
assignee:riccardobrasca
12-82269
12 days ago
13-26437
13 days ago
2-27612
2 days
24130 AntoineChambert-Loir
author:AntoineChambert-Loir
feat(GroupTheory/GroupAction/MultiplyPretransitive) : Multiple transivity property of the permutation group * The permutation group is pretransitive, is multiply pretransitive, and is preprimitive (for its natural action) * `Equiv.Perm.eq_top_if_isMultiplyPretransitive`: a subgroup of `Equiv.Perm α` which is `Nat.card α - 1` pretransitive is equal to `⊤`. --- - [x] depends on: #24167 - [x] depends on: #24117 - [x] depends on: #24107 - [x] depends on: #23962 - [x] depends on: #23386 - [ ] depends on: #23979 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra blocked-by-other-PR
label:t-algebra$
1573/6 Mathlib.lean,Mathlib/Algebra/Group/End.lean,Mathlib/GroupTheory/GroupAction/FixingSubgroup.lean,Mathlib/GroupTheory/GroupAction/Jordan.lean,Mathlib/GroupTheory/GroupAction/MultiplePrimitivity.lean,Mathlib/GroupTheory/GroupAction/MultipleTransitivity.lean,Mathlib/GroupTheory/GroupAction/Primitive.lean,Mathlib/GroupTheory/GroupAction/SubMulAction.lean,Mathlib/GroupTheory/GroupAction/SubMulAction/OfFixingSubgroup.lean 9 5 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] riccardobrasca
assignee:riccardobrasca
12-81407
12 days ago
12-81425
12 days ago
1-57991
1 day
25248 xcloudyunx
author:xcloudyunx
feat(Combinatorics/SimpleGraph): Add Subgraph.inclusion_edge_apply_coe and inclusion_edgeSet_apply_coe --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-combinatorics 12/0 Mathlib/Combinatorics/SimpleGraph/Subgraph.lean 1 1 ['github-actions'] nobody
12-76744
12 days ago
12-76745
12 days ago
12-76800
12 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$
91/17 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 16 ['alreadydone', 'erdOne', 'eric-wieser', 'github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'leanprover-community-mathlib4-bot', 'mathlib4-dependent-issues-bot'] erdOne
assignee:erdOne
12-72577
12 days ago
12-72595
12 days ago
55-19940
55 days
25238 Hagb
author:Hagb
feat(Tactic/ComputeDegree): add support for scalar multiplication with different types It would be able to deal with `a • (X : R[X])` where `a : S` is in a different type `S` with `[SMulZeroClass S R]`. --- - [x] depends on: #25237 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor 17/5 Mathlib/Tactic/ComputeDegree.lean,MathlibTest/ComputeDegree.lean 2 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
12-56734
12 days ago
12-81177
12 days ago
12-83080
12 days
24690 ScottCarnahan
author:ScottCarnahan
feat (Data.Prod): Reverse lexicographic order This PR implements the type synonym RevLex as a one-field structure, defines an order on products, and proves an order isomorphism with the Lex product with factors switched. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order WIP 141/0 Mathlib.lean,Mathlib/Data/Prod/RevLex.lean 2 4 ['ScottCarnahan', 'YaelDillies', 'github-actions'] YaelDillies
assignee:YaelDillies
12-50280
12 days ago
12-61973
12 days ago
19-33859
19 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
12-48292
12 days ago
16-14031
16 days ago
16-14015
16 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 7 ['Parcly-Taxel', 'YaelDillies', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant'] nobody
12-45087
12 days ago
12-45105
12 days ago
59-44919
59 days
25253 Ruben-VandeVelde
author:Ruben-VandeVelde
feat: add AlgHom.natCard_of_splits --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 21/7 Mathlib/FieldTheory/PrimitiveElement.lean,Mathlib/FieldTheory/Separable.lean,Mathlib/SetTheory/Cardinal/Finite.lean 3 1 ['github-actions'] nobody
12-43025
12 days ago
12-43107
12 days ago
12-43091
12 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
12-42970
12 days ago
13-18912
13 days ago
19-23308
19 days
24304 YaelDillies
author:YaelDillies
feat: continuous perfect pairings Define continuous perfect pairings using a Prop-valued typeclass `IsContPerfPair` on a bilinear pairing `p : M →ₗ[R] N →ₗ[R] R`, and a function to turn `p : M →ₗ[R] N →ₗ[R] R` + `p.IsContPerfPair` into `M ≃ₗ[R] (N →ₗ[R] R)`. The name `IsContPerfPair` is kept short because it shows up in lemma and definition names. Mathematically, there are many topological notions of perfect pairing: one per topology on `N →ₗ[R] R`/`N →L[R] R`. It is therefore better for `IsContPerfPair` not to require `p x` to be a homeo, and to instead extend it to new classes like `IsWeakTopPerfPair`, `IsCompactOpenPerfPair`, etc... whenever we need it to imply some reflexivity result for a particular norm on linear maps. There's also the question of continuity. Most applications need only continuity in either argument, but currently we are requiring continuity in both arguments simultaneously, ie as a map `M × N → R`. This is an easy way to ensure we get a map `N → M →L[R] R`. From Toric Co-authored-by: Andrew Yang --- `PerfectPairing` can be similarly refactored, but this should be a later PR. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) toric t-topology 71/0 Mathlib.lean,Mathlib/Topology/Algebra/Module/PerfectPairing.lean 2 8 ['ADedecker', 'YaelDillies', 'erdOne', 'github-actions', 'ocfnash'] ADedecker
assignee:ADedecker
12-34873
12 days ago
13-47395
13 days ago
47-42005
47 days
23426 idontgetoutmuch
author:idontgetoutmuch
G-Bundle and examples --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-differential-geometry awaiting-author 691/0 Mathlib/Topology/FiberBundle/Instances/GBundleDefs.lean,Mathlib/Topology/FiberBundle/Instances/Mobius.lean,Mathlib/Topology/FiberBundle/Instances/MobiusAsGBundle.lean 3 4 ['eric-wieser', 'idontgetoutmuch'] nobody
12-33132
12 days ago
23-45450
23 days ago
0-0
0 seconds
25179 YaelDillies
author:YaelDillies
feat: `#track_sorry`, a command to find usage of `sorry` `#track_sorry foo` returns a non-sorry-free declaration `bar` which `foo` depends on, if such `bar` exists. Such a command is a recurrent need of the community, see eg [here](https://leanprover.zulipchat.com/#narrow/channel/217875-Is-there-code-for-X.3F/topic/Hunting.20down.20axioms/with/495448595) most recently. From Toric Co-authored-by: Henrik Böving --- An alternative implementation was provided in [#Is there code for X? > ✔ Finding usages of `sorry` in external code @ 💬](https://leanprover.zulipchat.com/#narrow/channel/217875-Is-there-code-for-X.3F/topic/.E2.9C.94.20Finding.20usages.20of.20.60sorry.60.20in.20external.20code/near/430509619) by @kmill. I prefer the current one because it only prints something for uses of `sorry` and not the other three standard axioms. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) toric t-meta 71/0 Mathlib.lean,Mathlib/Util/TrackSorry.lean 2 11 ['YaelDillies', 'eric-wieser', 'github-actions', 'kmill'] nobody
12-33079
12 days ago
15-41894
15 days ago
15-41948
15 days
25257 Hagb
author:Hagb
feat(Mathlib/Algebra/Polynomial/Degree/Domain.lean): generalize `natDegree_smul` from `SMulWithZero` to `SMulZeroClass` as suggested by @eric-wieser in https://github.com/leanprover-community/mathlib4/pull/25237#discussion_r2111599865 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra
label:t-algebra$
4/3 Mathlib/Algebra/Polynomial/Degree/Domain.lean 1 1 ['github-actions'] nobody
12-26109
12 days ago
12-26109
12 days ago
12-26171
12 days
25261 hanwenzhu
author:hanwenzhu
feat(ProbabilityTheory): Conditional Jensen WIP cc @CoolRmal Co-authored-by: Yongxi Lin <97214596+CoolRmal@users.noreply.github.com> --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 27/0 test.lean 1 1 ['github-actions'] nobody
12-17195
12 days ago
12-17266
12 days ago
0-0
0 seconds
25262 Ruben-VandeVelde
author:Ruben-VandeVelde
chore: add missing deprecations From #23643, #23804, #24762, #24827, #24833, and #25016. --- Maybe for some of those there could be reasons to argue that a deprecation is not terribly useful, but adding them is so cheap that I don't think it's worth spending much time arguing about it. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 36/0 Mathlib/AlgebraicGeometry/IdealSheaf/Basic.lean,Mathlib/Analysis/SpecialFunctions/Complex/LogBounds.lean,Mathlib/Analysis/SpecialFunctions/MulExpNegMulSqIntegral.lean,Mathlib/GroupTheory/Perm/Finite.lean,Mathlib/GroupTheory/Perm/Support.lean,Mathlib/NumberTheory/NumberField/InfinitePlace/TotallyRealComplex.lean,Mathlib/RingTheory/Ideal/Operations.lean,Mathlib/RingTheory/MvPowerSeries/PiTopology.lean 8 1 ['github-actions'] nobody
12-15004
12 days ago
12-17260
12 days ago
12-17244
12 days
25251 YaelDillies
author:YaelDillies
chore: move pointed cones, proper cones Pointed cones too are a kind of algebraic cone. They therefore move to the new `Geometry.Convex.Cone` folder. In turn, this makes proper cones the primitive kind of topological/analytic cones, and therefore `Analysis.Convex.Cone.Proper` gets renamed to `Analysis.Convex.Cone.Basic`. The two sections about dual pointed cones and dual proper cones move to the existing `Analysis.Convex.Cone.InnerDual`. The READMEs about `Geometry.Convex.Cone` and `Analysis.Convex.Cone` get updated to reflect that the separation is non-topology vs topology, rather topology vs analysis. From Toric --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) file-removed toric large-import t-analysis 112/115 Mathlib.lean,Mathlib/Analysis/Convex/Cone/Basic.lean,Mathlib/Analysis/Convex/Cone/Closure.lean,Mathlib/Analysis/Convex/Cone/InnerDual.lean,Mathlib/Analysis/Convex/Cone/README.md,Mathlib/Geometry/Convex/Cone/Basic.lean,Mathlib/Geometry/Convex/Cone/Pointed.lean,Mathlib/Geometry/Convex/Cone/README.md 8 2 ['github-actions', 'leanprover-community-bot-assistant'] nobody
12-12573
12 days ago
12-20075
12 days ago
12-36173
12 days
25266 j-loreaux
author:j-loreaux
feat: add path component of the identity in a locally path connected topological group, as an open normal subgroup --- From [LeanOA](https://github.com/j-loreaux/LeanOA) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology 101/8 Mathlib.lean,Mathlib/Topology/Connected/PathComponentOne.lean,Mathlib/Topology/Connected/PathConnected.lean,Mathlib/Topology/Path.lean 4 1 ['github-actions'] nobody
12-7869
12 days ago
12-10701
12 days ago
12-11347
12 days
25271 YaelDillies
author:YaelDillies
feat: promote an `AlgEquiv` preserving `counit` and `comul` to a `BialgEquiv` From Toric --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) toric t-algebra
label:t-algebra$
38/24 Mathlib/Algebra/Algebra/Equiv.lean,Mathlib/Algebra/Algebra/Hom.lean,Mathlib/RingTheory/Bialgebra/Equiv.lean 3 1 ['github-actions'] nobody
12-6409
12 days ago
12-10058
12 days ago
12-10053
12 days
24131 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. --- - [x] depends on: #24167 - [x] depends on: #24117 - [x] depends on: #24107 - [x] depends on: #23962 - [x] depends on: #23386 - [ ] depends on: #23979 - [ ] depends on: #24130 - [ ] depends on: #24120 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-algebra blocked-by-other-PR
label:t-algebra$
2079/40 Mathlib.lean,Mathlib/Algebra/Group/End.lean,Mathlib/GroupTheory/GroupAction/FixingSubgroup.lean,Mathlib/GroupTheory/GroupAction/Jordan.lean,Mathlib/GroupTheory/GroupAction/MultiplePrimitivity.lean,Mathlib/GroupTheory/GroupAction/MultipleTransitivity.lean,Mathlib/GroupTheory/GroupAction/Primitive.lean,Mathlib/GroupTheory/GroupAction/SubMulAction.lean,Mathlib/GroupTheory/GroupAction/SubMulAction/OfFixingSubgroup.lean,Mathlib/SetTheory/Cardinal/Embedding.lean 10 8 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
12-317
12 days ago
12-3252
12 days ago
0-1323
22 minutes
25283 Brian-Nugent
author:Brian-Nugent
feat: regular local rings Adds regular local rings and proves they are integral domains. --- - [ ] depends on: #25280 - [ ] depends on: #25282 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra blocked-by-other-PR
label:t-algebra$
871/0 .vscode/settings.json,Mathlib.lean,Mathlib/RingTheory/EmbeddingDimension.lean,Mathlib/RingTheory/LocalRingDimension.lean,Mathlib/RingTheory/RegularLocalRing.lean 5 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
11-84684
11 days ago
11-84686
11 days ago
0-882
14 minutes
25282 Brian-Nugent
author:Brian-Nugent
feat: krull dimension facts for Noetherian local rings Proves that when modding out by a non-unit, the Krull dimension of a noetherian local ring drops by at most one. Also proves that the embedding dimension is an upper bound on the Krull dimension. --- - [ ] depends on: #25280 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra blocked-by-other-PR
label:t-algebra$
626/0 .vscode/settings.json,Mathlib.lean,Mathlib/RingTheory/EmbeddingDimension.lean,Mathlib/RingTheory/LocalRingDimension.lean 4 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
11-84683
11 days ago
11-84685
11 days ago
0-1566
26 minutes
25173 Timeroot
author:Timeroot
"Junk value" test file Add to MathlibTest a file that documents junk values of many functions, and explains some of their motivations and gotchas. --- Based on the conversation [on Zulip](https://leanprover.zulipchat.com/#narrow/channel/113488-general/topic/Documenting.20lean.20pitfalls.3A.20feedback.20requested/near/520155520). [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 362/2 Mathlib/Data/Nat/Find.lean,MathlibTest/Junk.lean 2 15 ['Timeroot', 'github-actions', 'plp127'] nobody
11-84537
11 days ago
15-59398
15 days ago
15-59382
15 days
25247 alreadydone
author:alreadydone
Projective contraction --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
160/31 Mathlib/Data/Finsupp/Defs.lean,Mathlib/LinearAlgebra/Contraction.lean,Mathlib/LinearAlgebra/Pi.lean,Mathlib/RingTheory/Finiteness/Finsupp.lean 4 1 ['github-actions'] nobody
11-79860
11 days ago
12-80718
12 days ago
0-30
30 seconds
24582 pechersky
author:pechersky
feat(GroupTheory/ArchimedeanDensely): Unique (ℤ ≃+o ℤ) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) - [x] depends on: #24580 t-order t-algebra
label:t-algebra$
44/0 Mathlib/Data/Int/Cast/Lemmas.lean,Mathlib/GroupTheory/ArchimedeanDensely.lean 2 5 ['eric-wieser', 'github-actions', 'mathlib4-dependent-issues-bot', 'pechersky'] nobody
11-65302
11 days ago
11-65375
11 days ago
15-28500
15 days
24412 pechersky
author:pechersky
feat(UniformSpace/Ultra/Constructions): IsUltraUniformity.{bot,top} --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-topology 29/0 Mathlib/Order/Filter/Bases/Basic.lean,Mathlib/Topology/UniformSpace/Defs.lean,Mathlib/Topology/UniformSpace/Ultra/Basic.lean,Mathlib/Topology/UniformSpace/Ultra/Constructions.lean 4 6 ['github-actions', 'pechersky', 'urkud'] urkud
assignee:urkud
11-64083
11 days ago
11-67293
11 days ago
36-64253
36 days
22919 plp127
author:plp127
feat(Data/Fintype/Pi): Make `Fintype` instance for `RelHom`s computable Makes the `Fintype` instance for rel homs computable. See this [Zulip](https://leanprover.zulipchat.com/#narrow/channel/113489-new-members/topic/Classical.20vs.20constructive.20logic.20in.20computation/near/496220816) message. --- - [x] depends on: #24748 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data awaiting-author 178/44 Mathlib/Combinatorics/SimpleGraph/Basic.lean,Mathlib/Combinatorics/SimpleGraph/Coloring.lean,Mathlib/Combinatorics/SimpleGraph/Maps.lean,Mathlib/Data/Fintype/CardEmbedding.lean,Mathlib/Data/Fintype/Pi.lean 5 29 ['IvanRenison', 'b-mehta', 'eric-wieser', 'fpvandoorn', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'plp127'] b-mehta
assignee:b-mehta
11-58021
11 days ago
11-58021
11 days ago
73-73341
73 days
25161 BoltonBailey
author:BoltonBailey
chore(Algebra/Squarefree/Basic): fix erw This PR addresses an instance of the `erw` linter in `Algebra/Squarefree/Basic` by adding a `squarefree_def` theorem and using this to isolate the implementation. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) tech debt t-algebra awaiting-author
label:t-algebra$
4/1 Mathlib/Algebra/Squarefree/Basic.lean 1 3 ['b-mehta', 'eric-wieser', 'github-actions'] nobody
11-57924
11 days ago
11-57924
11 days ago
4-35623
4 days
25239 YaelDillies
author:YaelDillies
refactor: redefine perfect pairings as a Prop-valued typeclass Redefine perfect pairings using a Prop-valued typeclass `IsPerfPair` on a bilinear pairing `p : M →ₗ[R] N →ₗ[R] R`, and a function to turn `p : M →ₗ[R] N →ₗ[R] R` + `p.IsPerfPair` into `M ≃ₗ[R] Dual R N`. The name `IsPerfPair` is kept short because it shows up in lemma and definition names. From Toric --- @ocfnash, do you like the direction this is going in? [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) toric t-algebra awaiting-CI
label:t-algebra$
277/164 Mathlib/LinearAlgebra/PerfectPairing/Basic.lean,Mathlib/LinearAlgebra/PerfectPairing/Restrict.lean,Mathlib/LinearAlgebra/RootSystem/Defs.lean,Mathlib/LinearAlgebra/RootSystem/Hom.lean,Mathlib/LinearAlgebra/RootSystem/IsValuedIn.lean,Mathlib/LinearAlgebra/RootSystem/OfBilinear.lean 6 10 ['YaelDillies', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'ocfnash'] nobody
11-45140
11 days ago
11-45157
11 days ago
1-235
1 day
25273 YaelDillies
author:YaelDillies
feat: `Finsupp.linearCombination MonoidAlgebra.of = id` From Toric --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-algebra
label:t-algebra$
8/1 Mathlib/Algebra/MonoidAlgebra/Defs.lean 1 4 ['YaelDillies', 'eric-wieser', 'github-actions'] nobody
11-40091
11 days ago
12-8231
12 days ago
12-8280
12 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 --- - [ ] depends on: #25291 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-convex-geometry toric blocked-by-other-PR 217/214 Mathlib/Analysis/Convex/Cone/Pointed.lean,Mathlib/Geometry/Convex/Cone/Basic.lean 2 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
11-37547
11 days ago
11-40576
11 days ago
0-690
11 minutes
25291 YaelDillies
author:YaelDillies
chore(Geometry/Convex/Cone/Basic): clean up Rename all the `ConvexCone`s in the file to `C`, `C₁`, `C₂`. Previously they were `S`, `T`, `K₁`, `K₂`. Make sure to tag all the relevant lemmas with `norm_cast`. Fix lemma names. Golf proofs. From Toric --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-convex-geometry toric 145/186 Mathlib/Analysis/Convex/Cone/Pointed.lean,Mathlib/Geometry/Convex/Cone/Basic.lean 2 1 ['github-actions'] nobody
11-36836
11 days ago
11-41271
11 days ago
11-41327
11 days
7300 ah1112
author:ah1112
feat: synthetic geometry This is adding synthetic geometry using Avigad's axioms and formalizing Euclid Book I, through the Pythagorean theorem. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-euclidean-geometry awaiting-author help-wanted 2661/0 Mathlib.lean,Mathlib/Geometry/Synthetic/Avigad/Axioms.lean,Mathlib/Geometry/Synthetic/Avigad/EuclidBookI.lean,Mathlib/Geometry/Synthetic/Avigad/Tactics.lean 4 72 ['ah1112', 'alreadydone', 'eric-wieser', 'github-actions', 'tb65536', 'urkud'] nobody
11-18588
11 days ago
502-85828
1 year ago
0-0
0 seconds
25290 linesthatinterlace
author:linesthatinterlace
feat: Low-level derivatives of lifts on `OneHom`, `MulHom` and `MonoidHom` --- - [ ] depends on: #25264 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra blocked-by-other-PR
label:t-algebra$
652/33 Mathlib/Algebra/Group/Equiv/Basic.lean,Mathlib/Algebra/Group/Hom/Basic.lean,Mathlib/Algebra/Group/Hom/Defs.lean 3 3 ['github-actions', 'linesthatinterlace', 'mathlib4-dependent-issues-bot'] nobody
11-9838
11 days ago
11-42240
11 days ago
0-762
12 minutes
22490 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. --- - [x] depends on: #22474 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory 160/0 Mathlib.lean,Mathlib/CategoryTheory/Functor/Derived/PointwiseRightDerived.lean 2 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
11-8730
11 days ago
11-8995
11 days ago
11-11016
11 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
11-7081
11 days ago
11-7081
11 days ago
11-25466
11 days
23161 mans0954
author:mans0954
feature(Data/Finset/RangeDistance): abs_sub_lt_of_mem_finset_range The distance between two elements of `Finset.range N` (i.e. absolute value of the difference as integers) is less than `N`. A lemma I found useful for something I was working on, so sharing here in case it's of wider interest. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data 30/0 Mathlib.lean,Mathlib/Algebra/Order/Group/Unbundled/Abs.lean,Mathlib/Data/Finset/RangeDistance.lean 3 4 ['fbarroero', 'github-actions', 'mans0954'] ericrbg
assignee:ericrbg
10-82258
10 days ago
81-2744
2 months ago
81-2735
81 days
15412 mans0954
author:mans0954
feat(Order/ScottContinuity): Scott continuity on product spaces Some further results on Scott Continuity: - `scottContinuous_iff_map_sSup`: `f` is Scott continuous if and only if it commutes with `sSup` on directed sets - `ScottContinuous_prod_of_ScottContinuous`: `f` is Scott continuous on a product space if it is Scott continuous in each variable - `ScottContinuousOn.inf₂`: For complete linear orders, the meet operation is Scott continuous --- - [x] depends on: #13201 - I think this is due to the move of the definition of Scott Continuity into its own file rather than a hard dependency. - [x] depends on: #19150 - [x] depends on: #19222 - [x] depends on:#20254 - [x] depends on: #21493 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-order 78/5 Mathlib/Order/ScottContinuity.lean 1 n/a ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
10-82102
10 days ago
unknown
unknown
25170 eric-wieser
author:eric-wieser
refactor: make basis computable I claim that in the long run, `Basis.repr` should be a `DFinsupp` not `Finsupp`, so that it is computable. To make this change incrementally, we can store a `DFinsupp` internally today, and keep `repr` and `ofRepr` working with finsupp. This at least would allow building a large basis object, and then using `repr'` to compute with it. The cost of this intermediate state is a loss of many defeqs. --- - [ ] depends on: #25166 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-algebra
label:t-algebra$
66/21 Mathlib/LinearAlgebra/Basis/Basic.lean,Mathlib/LinearAlgebra/Basis/Defs.lean,Mathlib/LinearAlgebra/FreeModule/Basic.lean 3 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
10-73673
10 days ago
11-38671
11 days ago
0-0
0 seconds
20704 winstonyin
author:winstonyin
feat: existence of local flows of vector fields I formalise the existence theorem for local flows of time-dependent vector fields (`IsPicardLindelof.exists_forall_mem_closedBall_eq_hasDerivWithinAt`). Currently, if we wish to show the existence of a family of integral curves indexed by their initial conditions, it is necessary to prove the hypotheses of the vector field (Lipschitz continuity within a closed ball, etc.), centred around each of these initial conditions. I have refactored the current proof of the Picard-Lindelöf theorem to allow the initial point to be different from the point about which the hypotheses on the vector field are stated. This way, integral curves and flows are treated on equal footing. Credits going to the original author @urkud, I have completely rewritten the file to accommodate different design choices. Many of the proof steps are nevertheless inspired by Yury's formalisation. * The `PicardLindelof` data structure is removed entirely. It merely bundles the non-Prop arguments into itself. Although it simplifies the assumptions in subsequent proofs, it obscures the (in)dependence on the relevant constants in the type description of theorems. Since `IsPicardLindelof` is already a public facing structure, we should also simply use it internally, without any loss. * In particular, I remove the completely superficial dependence of `FunSpace` on the `PicardLindelof` structure. * `FunSpace` no longer specifies the initial condition. It only needs the initial point to lie in a closed ball (which will be the domain of the local flow). * I avoid defining new non-Prop things that are only used in the proof steps, such as the current `vComp` and `tDist`. The proofs are a little longer as a result, but they are also more readable. * I place all private (i.e. only internally used) theorems under the namespace `FunSpace`, to guide users to the proper theorems in the public API. This is part of my effort to show that the solution to an ODE depends smoothly on the initial condition, or on parameters of the ODE. This is in turn needed for many results about manifolds, such as the fact that $C^1$ vector fields on compact manifolds always have global integral curves (or global flows). I especially welcome any suggestions to rename lemmas or define new structures to simplify the statements. I'm happy to write up the proof in LaTeX as well, if it's going to help reviewers. - [x] depends on: #20696 - [x] depends on: #20731 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-dynamics t-analysis 562/360 Mathlib/Algebra/Order/Group/Abs.lean,Mathlib/Analysis/Normed/Group/Basic.lean,Mathlib/Analysis/ODE/PicardLindelof.lean,Mathlib/Geometry/Manifold/IntegralCurve/ExistUnique.lean,docs/1000.yaml,docs/undergrad.yaml 6 27 ['github-actions', 'grunweg', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'michaellee94', 'winstonyin'] grunweg
assignee:grunweg
10-44673
10 days ago
10-48602
10 days ago
77-37721
77 days
25062 erdOne
author:erdOne
feat(Algebra/MvPolynomial): nilpotents and units --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
113/0 Mathlib.lean,Mathlib/Algebra/MvPolynomial/Nilpotent.lean,Mathlib/Data/Finsupp/Basic.lean 3 8 ['alreadydone', 'erdOne', 'eric-wieser', 'github-actions'] nobody
10-22453
10 days ago
19-70059
19 days ago
19-70108
19 days
24689 chrisflav
author:chrisflav
feat(Topology): compact open covered sets This is used to define the fpqc topology for schemes. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) maintainer-merge t-algebraic-geometry t-topology 219/0 Mathlib.lean,Mathlib/Data/Set/Sigma.lean,Mathlib/Topology/Compactness/Compact.lean,Mathlib/Topology/Sets/CompactOpenCovered.lean,Mathlib/Topology/Sets/Opens.lean,Mathlib/Topology/Spectral/Prespectral.lean 6 5 ['chrisflav', 'erdOne', 'github-actions', 'leanprover-community-bot-assistant'] nobody
10-5014
10 days ago
10-5399
10 days ago
31-65140
31 days
25313 jt496
author:jt496
feat(SimpleGraph/FiveWheelLike): add the Andrásfai-Erdős-Sós theorem Add the Andrásfai-Erdős-Sós theorem `colorable_of_cliqueFree_lt_minDegree` which says that an `r + 1`-cliquefree graph `G` with sufficiently large minimum degree is `r`-colorable. Co-authored-by: Lian Bremner Tattersall --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-combinatorics 307/4 Mathlib/Combinatorics/SimpleGraph/FiveWheelLike.lean 1 1 ['github-actions'] nobody
9-73651
9 days ago
10-35687
10 days ago
10-35738
10 days
25324 eric-wieser
author:eric-wieser
feat: more functorial results about DFinsupp --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) [#mathlib4 > Equiv.cast for structures @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Equiv.2Ecast.20for.20structures/near/521390935) WIP 140/15 Mathlib/Data/DFinsupp/Defs.lean,Mathlib/LinearAlgebra/DFinsupp.lean 2 1 ['github-actions'] nobody
9-69236
9 days ago
9-69769
9 days ago
0-0
0 seconds
21950 erdOne
author:erdOne
feat(NumberTheory/Padics): the completion of `ℚ` at a finite place is `ℚ_[p]` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-number-theory 253/1 Mathlib.lean,Mathlib/Algebra/GroupWithZero/WithZero.lean,Mathlib/NumberTheory/Padics/HeightOneSpectrum.lean,Mathlib/NumberTheory/Padics/PadicNumbers.lean,Mathlib/Topology/Algebra/Valued/WithVal.lean,Mathlib/Topology/Algebra/WithZeroMulInt.lean,Mathlib/Topology/Algebra/WithZeroTopology.lean 7 22 ['Ruben-VandeVelde', 'erdOne', 'github-actions', 'leanprover-community-bot-assistant', 'pechersky', 'smmercuri', 'xroblot'] nobody
9-68894
9 days ago
9-68894
9 days ago
51-21490
51 days
25322 thorimur
author:thorimur
style: use simplex notation (`⦋n⦌`) where possible `StandardSimplex.mk n` is replaced with `⦋n⦌` where possible (except in notation and macros, which are left untouched). This includes opening `Simplicial` in two files. Also, outdated and unused `local notation` `[n]` for `StandardSimplex.mk n` is removed. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology 38/39 Mathlib/AlgebraicTopology/CechNerve.lean,Mathlib/AlgebraicTopology/MooreComplex.lean,Mathlib/AlgebraicTopology/SimplexCategory/Basic.lean,Mathlib/AlgebraicTopology/SimplicialObject/Basic.lean,Mathlib/AlgebraicTopology/SimplicialSet/Coskeletal.lean,Mathlib/AlgebraicTopology/SimplicialSet/NerveAdjunction.lean,Mathlib/AlgebraicTopology/SimplicialSet/StdSimplex.lean 7 1 ['github-actions'] nobody
9-65931
9 days ago
9-76510
9 days ago
9-76563
9 days
24173 YaelDillies
author:YaelDillies
feat: the composition of open relations is open [Zulip](https://leanprover.zulipchat.com/#narrow/channel/217875-Is-there-code-for-X.3F/topic/.60IsOpen.60.20and.20.60compRel.60) --- - [ ] depends on: #23181 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology blocked-by-other-PR 50/1 Mathlib/Topology/Bases.lean,Mathlib/Topology/UniformSpace/Basic.lean,Mathlib/Topology/UniformSpace/Defs.lean 3 4 ['ADedecker', 'Komyyy', 'github-actions', 'mathlib4-dependent-issues-bot'] nobody
9-64807
9 days ago
51-17122
1 month ago
0-82106
22 hours
25288 robertmaxton42
author:robertmaxton42
feat(CategoryTheory): generalize `Discrete` to arbitrary morphism levels Using an unused `let`, add an 'anchor' to the definition of `Discrete`, allowing it to carry a second universe level that is then used to permit discrete categories to live in any `Cat.{v, u}`. (This trick was borrowed from the code of `ULiftHom`.) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory 38/32 Mathlib/CategoryTheory/Bicategory/LocallyDiscrete.lean,Mathlib/CategoryTheory/Discrete/Basic.lean,Mathlib/CategoryTheory/IsConnected.lean 3 2 ['github-actions', 'joelriou'] nobody
9-43233
9 days ago
9-81773
9 days ago
0-0
0 seconds
24373 YaelDillies
author:YaelDillies
refactor: golf `modularCharacter` ... using the lessons learned from `distribHaarChar`. Unfortunately, the two setups can't quite be unified because we are lacking an additive version of `MulDistribMulAction`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-measure-probability awaiting-CI 82/48 Mathlib/MeasureTheory/Group/MeasurableEquiv.lean,Mathlib/MeasureTheory/Group/Measure.lean,Mathlib/MeasureTheory/Group/ModularCharacter.lean,Mathlib/MeasureTheory/Integral/Bochner/Basic.lean,Mathlib/MeasureTheory/Measure/Haar/Unique.lean 5 2 ['github-actions', 'leanprover-community-bot-assistant'] nobody
9-42364
9 days ago
9-42388
9 days ago
0-0
0 seconds
24490 dagurtomas
author:dagurtomas
feat(CategoryTheory): transport symmetric monoidal structure along equivalence --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory 89/0 Mathlib.lean,Mathlib/CategoryTheory/Monoidal/Braided/Basic.lean,Mathlib/CategoryTheory/Monoidal/Braided/Transport.lean 3 6 ['dagurtomas', 'github-actions', 'joelriou', 'kckennylau', 'leanprover-community-bot-assistant'] nobody
9-30633
9 days ago
9-30693
9 days ago
21-74160
21 days
24439 mariainesdff
author:mariainesdff
feat(Data/Nat/Factorial/NatCast): add natCast_factorial_of_isNilpotent 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 delegated
label:t-algebra$
32/2 Mathlib/Data/Nat/Factorial/NatCast.lean 1 3 ['b-mehta', 'github-actions', 'mariainesdff'] ocfnash
assignee:ocfnash
9-21321
9 days ago
41-27829
1 month ago
42-15186
42 days
25315 ocfnash
author:ocfnash
feat: add `simp` to lemma `Fin.coe_ofNat_eq_mod` One consequence is that `simp` can now prove things like this: ```lean example : (3 : Fin 10).val = 3 := by simp example : (4 : Fin 10).val = 4 := by simp example : (5 : Fin 10).val = 5 := by simp ``` previously this only this only worked up to `(2 : Fin 10).val = 2` (via lemmas like `Fin.val_two`). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data 32/28 Archive/Imo/Imo2024Q5.lean,Mathlib/AlgebraicTopology/DoldKan/Faces.lean,Mathlib/Analysis/CStarAlgebra/SpecialFunctions/PosPart.lean,Mathlib/Data/Fin/Basic.lean,Mathlib/Data/Fin/Parity.lean,Mathlib/Data/Fin/Rev.lean,Mathlib/GroupTheory/CommutingProbability.lean,Mathlib/GroupTheory/Perm/Fin.lean,Mathlib/RingTheory/ChainOfDivisors.lean,MathlibTest/matrix.lean 10 25 ['b-mehta', 'eric-wieser', 'github-actions', 'leanprover-bot', 'mattrobball', 'ocfnash'] nobody
9-18565
9 days ago
10-11743
10 days ago
10-11733
10 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 9 ['YaelDillies', 'erdOne', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant'] nobody
9-11474
9 days ago
9-11493
9 days ago
12-10225
12 days
25284 alreadydone
author:alreadydone
feat(LinearAlgebra/Contraction): bijectivity of `dualTensorHom` + generalize to CommSemiring --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
168/44 Mathlib/Data/Finsupp/Defs.lean,Mathlib/LinearAlgebra/Contraction.lean,Mathlib/LinearAlgebra/Pi.lean,Mathlib/LinearAlgebra/Trace.lean,Mathlib/RingTheory/Finiteness/Finsupp.lean 5 5 ['alreadydone', 'eric-wieser', 'github-actions', 'leanprover-bot'] nobody
8-77320
8 days ago
11-79692
11 days ago
11-79677
11 days
25078 loefflerd
author:loefflerd
feat(NumberTheory/ModularForms): GL(2, R) action preserves holomorphy Show that the slash action of negative-determinant matrices preserves holomorphic functions. --- - [x] depends on: #25028 - [x] depends on: #24740 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-number-theory 58/19 Mathlib/Analysis/Complex/UpperHalfPlane/Manifold.lean,Mathlib/NumberTheory/ModularForms/Basic.lean 2 5 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
8-38192
8 days ago
11-30057
11 days ago
11-30259
11 days
25343 plp127
author:plp127
docs(Topology/Perfect): Mention dense-in-itself The file `Mathlib/Topology/Perfect` defines a "nonstandard" predicate `Preperfect C` to mean that every point of `C` is an accumulation point of `C`. This property already has a name, it is called [dense-in-itself](https://en.wikipedia.org/wiki/Dense-in-itself). This PR adds this name to the docs. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology documentation 7/7 Mathlib/Topology/Perfect.lean 1 1 ['github-actions'] nobody
8-27307
8 days ago
8-27385
8 days ago
8-27370
8 days
24777 joelriou
author:joelriou
feat(CategoryTheory): abstract argument for the stability under transfinite compositions If a class of morphisms is multiplicative, respects isomorphisms and is stable under filtered colimits, then it is stable under transfinite compositions. (This simplifies the proof in the case of monomorphisms in Grothendieck abelian categories, for isomorphisms, and in #23282, we shall apply this to monomorphisms in `Type`.) --- - [x] depends on: #24773 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-category-theory 122/116 Mathlib/CategoryTheory/Abelian/GrothendieckAxioms/Colim.lean,Mathlib/CategoryTheory/Abelian/GrothendieckCategory/EnoughInjectives.lean,Mathlib/CategoryTheory/Abelian/GrothendieckCategory/Monomorphisms.lean,Mathlib/CategoryTheory/MorphismProperty/Limits.lean,Mathlib/CategoryTheory/MorphismProperty/TransfiniteComposition.lean 5 12 ['callesonne', 'github-actions', 'joelriou', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
8-11882
8 days ago
9-4698
9 days ago
21-28102
21 days
25140 wwylele
author:wwylele
feat: Hahn embedding theorem This proves [Hahn embedding theorem](https://en.wikipedia.org/wiki/Hahn_embedding_theorem), one among the 1000+ theorems project. This is still in early draft, which is why I put it in a throw-away folder. I'll gradually clean up code, put them to the right places, and PR small components. The proof roughly follows the ones in the following literature - Hausner, M.; Wendel, J.G. (1952), "Ordered vector spaces", Proceedings of the American Mathematical Society, 3 (6): 977–982, [doi](https://en.wikipedia.org/wiki/Doi_(identifier)):[10.1090/S0002-9939-1952-0052045-1](https://doi.org/10.1090%2FS0002-9939-1952-0052045-1) - Clifford, A.H. (1954), "Note on Hahn's Theorem on Ordered Abelian Groups", Proceedings of the American Mathematical Society, 5 (6): 860–863, [doi](https://en.wikipedia.org/wiki/Doi_(identifier)):[10.2307/2032549](https://doi.org/10.2307%2F2032549), [JSTOR](https://en.wikipedia.org/wiki/JSTOR_(identifier)) [2032549](https://www.jstor.org/stable/2032549) --- - [ ] depends on: #25190 - [ ] depends on: #25168 - [ ] depends on: #25157 - [ ] depends on: #25144 - [ ] depends on: #25338 - [ ] depends on: #25348 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR WIP 3395/0 Mathlib/HahnEmbedding/ArchimedeanClass.lean,Mathlib/HahnEmbedding/ArchimedeanSubgroup.lean,Mathlib/HahnEmbedding/Divisible.lean,Mathlib/HahnEmbedding/Hahn.lean,Mathlib/HahnEmbedding/LinearPMap.lean,Mathlib/HahnEmbedding/Main.lean,Mathlib/HahnEmbedding/Misc.lean,Mathlib/HahnEmbedding/RealEmbed.lean,docs/1000.yaml 9 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
8-8366
8 days ago
15-15816
15 days ago
0-0
0 seconds
24514 b-mehta
author:b-mehta
chore(Int/GCD): use fuel in xgcd Modify the definition of xgcd to use fuel recursion, to allow it to be reduced in the kernel. As a consequence, this means the evaluation of field operations in ZMod p become provable by `rfl` and `decide`. Zulip discussion: https://leanprover.zulipchat.com/#narrow/channel/270676-lean4/topic/opaque.20recursion.20definitions.20break.20mergeSort.20decidability --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data 44/22 Mathlib/Data/Int/GCD.lean 1 4 ['b-mehta', 'eric-wieser', 'github-actions', 'nomeata', 'urkud'] nobody
7-84218
7 days ago
39-19437
1 month ago
39-19489
39 days
24543 pfaffelh
author:pfaffelh
feat (Topology/Compactness/CompactSystem): Set system of finite unions of sets in a compact system is again a compact system feat (Topology/Compactness/CompactSystem): The set system of finite unions of sets in a compact system is a compact system A compact system is a set system with the following property: If all finite intersections of a sequence in the set system is non-empty, the countable intersection is not empty. Starting with a compact system, consider the finite unions of sets in the copact system. Such sets again form a compact system (`IsCompactSystem.union.isCompactSystem`). --- - [x] depends on: #24541 - [x] depends on: #24542 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-topology blocked-by-other-PR 431/2 Mathlib/Topology/Compactness/CompactSystem.lean 1 4 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
7-82487
7 days ago
7-82487
7 days ago
0-1830
30 minutes
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
7-62144
7 days ago
8-71866
8 days ago
8-71857
8 days
24065 kim-em
author:kim-em
chore: script to give topological sort of modules This script is not useful by itself: it just gives a topological sort of Mathlib's import graph. But I've several times found it useful when I want to modify many files systematically with minimal rebuilding: just work backwards through the list. awaiting-author 96/0 scripts/README.md,scripts/topological_sort.py 2 5 ['github-actions', 'jcommelin', 'kim-em'] jcommelin
assignee:jcommelin
7-49448
7 days ago
7-49448
7 days ago
48-7769
48 days
24320 robin-carlier
author:robin-carlier
chore(Category/Theory/Whiskering): tag `[reassoc]` some lemmas about isoWhisker Using the extension of `reassoc` to equality of isomorphisms, tags some lemmas in `CategoryTheory.Whiskering` with this new version of the attribute. --- - [ ] depends on: #24303 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory 179/11 Mathlib.lean,Mathlib/CategoryTheory/Whiskering.lean,Mathlib/Tactic.lean,Mathlib/Tactic/CategoryTheory/IsoReassoc.lean,Mathlib/Tactic/CategoryTheory/Reassoc.lean,MathlibTest/CategoryTheory/Reassoc.lean 6 5 ['github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'robin-carlier'] nobody
7-47673
7 days ago
7-47694
7 days ago
7-52796
7 days
23500 DrLSimon
author:DrLSimon
feat(MeasureTheory/Decomposition): link the clipped sub of positive measures to Jordan decomposition This introduces a new file `Mathlib/MeasureTheory/Decomposition/JordanSub.lean` which develops the Jordan decomposition of the signed measure `μ.toSignedMeasure - ν.toSignedMeasure` for finite measures `μ` and `ν`, expressing it as the pair `(μ - ν, ν - μ)` of mutually singular finite measures. The key tool is the Hahn decomposition theorem, which yields a measurable partition of the space where `μ ≥ ν` and `ν ≥ μ`. Some basic results of `VectorMeasure` are also provided such as `restrict_neg`, `restrict_sub` `restrict_add_restrict_compl` and `Measure.toSignedMeasure_le_iff` within the `JordanSub.lean` file. They could be moved to another more central place (I guess `VectorMeasure/Basic.lean`). Similarly, `Measure.sub_zero` could go to `Sub.lean`. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-measure-probability 209/2 Mathlib.lean,Mathlib/MeasureTheory/Measure/Decomposition/Hahn.lean,Mathlib/MeasureTheory/Measure/Sub.lean,Mathlib/MeasureTheory/VectorMeasure/Basic.lean,Mathlib/MeasureTheory/VectorMeasure/Decomposition/JordanSub.lean 5 132 ['DavidLedvinka', 'DrLSimon', 'EtienneC30', 'github-actions', 'grunweg', 'urkud'] EtienneC30
assignee:EtienneC30
7-44161
7 days ago
7-44161
7 days ago
29-62586
29 days
23431 JovanGerb
author:JovanGerb
feat: Imo2020 q6 I formalized IMO2020 Q6. I followed the solution that I found when I was marticipating in the exam. I used the statement formalization that was given by @jsm28. Some lemmas should be added to mathlib itself instead of the IMO2020Q6 file. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) IMO 378/0 Archive.lean,Archive/Imo/Imo2020Q6.lean 2 2 ['github-actions', 'jsm28'] nobody
7-36807
7 days ago
72-26314
2 months ago
0-0
0 seconds
25327 YaelDillies
author:YaelDillies
feat: `F.obj M` is a commutative monoid object if `M` is From Toric --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) toric 11/3 Mathlib/CategoryTheory/Monoidal/CommMon_.lean,Mathlib/CategoryTheory/Monoidal/Mon_.lean 2 1 ['github-actions'] nobody
7-35334
7 days ago
9-34472
9 days ago
9-34465
9 days
24614 JovanGerb
author:JovanGerb
chore: rename field `inf` to `min` in `Lattice` As suggested by @eric-wieser, this PR renames the `sup` and `inf` fields in `Lattice` to `max` and `min`. This means that we now can extend `Lattice` and `LinearOrder` simultaneously without ending up with duplicate fields. This should be implemented in a future PR for existing classes like `CompleteLinearOrder`. [Zulip discussion](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/.60sup.60.2F.60inf.60.20or.20.60max.60.2F.60min.60.20for.20set.20interval.20lemmas.3F) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order awaiting-author 179/185 Mathlib/Algebra/Field/Subfield/Basic.lean,Mathlib/Algebra/Group/Subgroup/Lattice.lean,Mathlib/Algebra/Group/Submonoid/Basic.lean,Mathlib/Algebra/Group/Subsemigroup/Basic.lean,Mathlib/Algebra/Lie/Subalgebra.lean,Mathlib/Algebra/Module/Submodule/Lattice.lean,Mathlib/Algebra/Order/Kleene.lean,Mathlib/Algebra/Order/Ring/Idempotent.lean,Mathlib/Algebra/Ring/Subring/Basic.lean,Mathlib/Algebra/Ring/Subsemiring/Basic.lean,Mathlib/Algebra/Tropical/Lattice.lean,Mathlib/AlgebraicGeometry/IdealSheaf/Basic.lean,Mathlib/Analysis/BoxIntegral/Box/Basic.lean,Mathlib/Analysis/BoxIntegral/Partition/Basic.lean,Mathlib/Analysis/Convex/SimplicialComplex/Basic.lean,Mathlib/Analysis/Normed/Group/Seminorm.lean,Mathlib/Analysis/NormedSpace/ENormedSpace.lean,Mathlib/Analysis/NormedSpace/MStructure.lean,Mathlib/Analysis/Seminorm.lean,Mathlib/CategoryTheory/Groupoid/Subgroupoid.lean,Mathlib/CategoryTheory/Sites/Coverage.lean,Mathlib/CategoryTheory/Sites/Grothendieck.lean,Mathlib/CategoryTheory/Sites/Pretopology.lean,Mathlib/CategoryTheory/Sites/Sieves.lean,Mathlib/CategoryTheory/Subobject/Lattice.lean,Mathlib/CategoryTheory/Subpresheaf/Basic.lean,Mathlib/Combinatorics/Digraph/Basic.lean,Mathlib/Combinatorics/SimpleGraph/Basic.lean,Mathlib/Combinatorics/SimpleGraph/Subgraph.lean,Mathlib/Computability/Reduce.lean,Mathlib/Data/DFinsupp/Order.lean,Mathlib/Data/Finset/Lattice/Basic.lean,Mathlib/Data/Finsupp/Order.lean,Mathlib/Data/Multiset/UnionInter.lean,Mathlib/Data/Nat/PartENat.lean,Mathlib/Data/PEquiv.lean,Mathlib/Data/Real/Basic.lean,Mathlib/Data/Semiquot.lean,Mathlib/Data/Set/Basic.lean,Mathlib/Data/Setoid/Basic.lean,Mathlib/Data/Sum/Lattice.lean,Mathlib/Dynamics/Circle/RotationNumber/TranslationNumber.lean,Mathlib/Geometry/Convex/Cone/Basic.lean,Mathlib/Geometry/Manifold/ChartedSpace.lean,Mathlib/GroupTheory/Congruence/Defs.lean,Mathlib/LinearAlgebra/AffineSpace/AffineSubspace/Defs.lean,Mathlib/LinearAlgebra/LinearPMap.lean,Mathlib/MeasureTheory/Function/AEEqFun.lean,Mathlib/MeasureTheory/Function/SimpleFunc.lean,Mathlib/ModelTheory/Substructures.lean,Mathlib/Order/BooleanSubalgebra.lean,Mathlib/Order/Booleanisation.lean,Mathlib/Order/CompleteLattice/Defs.lean,Mathlib/Order/Concept.lean,Mathlib/Order/ConditionallyCompleteLattice/Defs.lean,Mathlib/Order/Copy.lean,Mathlib/Order/Filter/Basic.lean,Mathlib/Order/Filter/Germ/Basic.lean,Mathlib/Order/FixedPoints.lean,Mathlib/Order/GaloisConnection/Basic.lean,Mathlib/Order/Heyting/Basic.lean,Mathlib/Order/Hom/Order.lean,Mathlib/Order/Ideal.lean,Mathlib/Order/Interval/Basic.lean,Mathlib/Order/Lattice.lean,Mathlib/Order/Partition/Finpartition.lean,Mathlib/Order/PropInstances.lean,Mathlib/Order/Sublattice.lean,Mathlib/Order/WithBot.lean,Mathlib/Probability/Process/Filtration.lean,Mathlib/RingTheory/Congruence/Basic.lean,Mathlib/RingTheory/Finiteness/Small.lean,Mathlib/RingTheory/NonUnitalSubring/Basic.lean,Mathlib/RingTheory/NonUnitalSubsemiring/Basic.lean,Mathlib/RingTheory/TwoSidedIdeal/Lattice.lean,Mathlib/RingTheory/UniqueFactorizationDomain/FactorSet.lean,Mathlib/RingTheory/Valuation/ValuationSubring.lean,Mathlib/Topology/Algebra/Group/GroupTopology.lean,Mathlib/Topology/Category/TopCat/OpenNhds.lean,Mathlib/Topology/LocallyFinsupp.lean,Mathlib/Topology/MetricSpace/BundledFun.lean,Mathlib/Topology/UniformSpace/Basic.lean 82 13 ['JovanGerb', 'bryangingechen', 'eric-wieser', 'github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'leanprover-community-mathlib4-bot'] nobody
7-31740
7 days ago
7-39051
7 days ago
1-85670
1 day
22069 Raph-DG
author:Raph-DG
feat(LinearMap): Added lemmas relating kernels of linear maps to Submodule.map Added the lemma ne_map_or_ne_kernel_inter_of_lt stating that if A < B as submodules, then for any linear map f, `ker f ⊓ A ≠ ker f ⊓ B ∨ Submodule.map f A ≠ Submodule.map f B`. We also prove the corollaries ker_inter_mono_of_map_eq and map_mono_of_ker_inter_eq. Co-authored-by: Raphael Douglas Giles (raphaeldouglasgiles@gmail.com) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra
label:t-algebra$
30/0 Mathlib/LinearAlgebra/Span/Basic.lean 1 21 ['Paul-Lez', 'Raph-DG', 'github-actions', 'j-loreaux', 'mattrobball'] mattrobball
assignee:mattrobball
7-31078
7 days ago
7-31078
7 days ago
109-70769
109 days
25358 YaelDillies
author:YaelDillies
chore: more shortcut instances for `ℤ` Currently, some of those instances are inferred from `Int.instNormedCommRing : NormedCommRing ℤ` once one imports `Mathlib.Analysis.Normed.Ring.Lemmas`. Among other things, this confuses `#min_imports`, which then invariably reports that `Mathlib.Analysis.Normed.Ring.Lemmas` is used. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra easy
label:t-algebra$
16/5 Mathlib/Algebra/Ring/Int/Defs.lean,Mathlib/NumberTheory/LegendreSymbol/GaussEisensteinLemmas.lean,Mathlib/NumberTheory/Zsqrtd/QuadraticReciprocity.lean 3 4 ['eric-wieser', 'github-actions', 'leanprover-bot'] nobody
7-29639
7 days ago
7-38392
7 days ago
7-39164
7 days
22052 FLDutchmann
author:FLDutchmann
feat(NumberTheory/SelbergSieve): define Lambda-squared sieves and prove important properties This PR: * Defines lambda-squared sieves. * Proves they are upper bound sieves. * Proves that the corresponding main sum is a quadratic form. --- - [x] depends on: #21880 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis t-number-theory awaiting-author 250/3 Mathlib/NumberTheory/SelbergSieve.lean 1 18 ['AlexKontorovich', 'Ruben-VandeVelde', 'github-actions', 'grunweg', 'jcommelin', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
7-25818
7 days ago
7-25818
7 days ago
61-33984
61 days
5897 eric-wieser
author:eric-wieser
feat: add a `MonadError` instance for `ContT` We already have a `MonadExcept` instance; this promotes it to `MonadError`. Note the issue with the existing `MonadExcept` instance still applies. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta awaiting-author 16/0 Mathlib/Control/Monad/Cont.lean 1 21 ['Vierkantor', 'YaelDillies', 'eric-wieser', 'github-actions', 'kmill'] nobody
6-70661
6 days ago
326-52157
10 months ago
339-53816
339 days
25383 sgouezel
author:sgouezel
feat: continuity statements for the bundle of continuous linear maps The continuity statements I am adding are counterparts of already existing ones for smooth maps. Also solve a TODO by dropping the type synonym `Bundle.ContinuousLinearMap`. It was useful a long time ago when the topology on the fibers was built using the norm on the model space. This is not the case since we've endowed all spaces of continuous linear maps on topological vector spaces with the topology of uniform convergence on bounded sets. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology 274/29 Mathlib/Analysis/Normed/Operator/BoundedLinearMaps.lean,Mathlib/Data/Bundle.lean,Mathlib/Geometry/Manifold/VectorBundle/Hom.lean,Mathlib/Topology/VectorBundle/Hom.lean 4 1 ['github-actions'] nobody
6-46150
6 days ago
6-46371
6 days ago
6-46356
6 days
25186 riccardobrasca
author:riccardobrasca
feat: add `isPrincipalIdealRing_of_isPrincipal_of_lt_or_isPrincipal_of_mem_primesOver_of_mem_Icc` The standard technique to prove that `𝓞 K` is principal in the Galois case. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-number-theory 45/9 Mathlib/NumberTheory/NumberField/ClassNumber.lean 1 14 ['faenuccio', 'github-actions', 'riccardobrasca'] nobody
6-37000
6 days ago
15-29033
15 days ago
15-29036
15 days
23970 AntoineChambert-Loir
author:AntoineChambert-Loir
feat(GroupTheory/GroupAction/SubMulAction/OfFixingSubgroup): action of the fixing Subgroup on the complement of a set Introduce the `SubMulAction` of a `fixingSubgroup` of a subset on the complement of that set. Develop relations between these and `SubMulAction` of stabilizers. --- - [x] depends on: #23386 - [x] depends on: #23962 - [x] depends on: #24107 - [x] depends on: #24117 - [x] depends on: #24167 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra delegated
label:t-algebra$
449/4 Mathlib.lean,Mathlib/Algebra/Group/End.lean,Mathlib/GroupTheory/GroupAction/FixingSubgroup.lean,Mathlib/GroupTheory/GroupAction/MultipleTransitivity.lean,Mathlib/GroupTheory/GroupAction/SubMulAction.lean,Mathlib/GroupTheory/GroupAction/SubMulAction/OfFixingSubgroup.lean 6 29 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib-bors', 'mathlib4-dependent-issues-bot', 'riccardobrasca'] riccardobrasca
assignee:riccardobrasca
6-35345
6 days ago
6-35345
6 days ago
13-15466
13 days
24480 mariainesdff
author:mariainesdff
feat(RingTheory/DividedPowers/SubPDIdeal): add SubDPIdeal Let `A` be a commutative (semi)ring and let `I` be an ideal of `A` with a divided power structure `hI`. A subideal `J` of `I` is a *sub-dp-ideal* of `(I, hI)` if, for all `n ∈ ℕ > 0` and all `x ∈ J`, `hI.dpow n x ∈ J`. The "TODOs" listed on the file docstring have been formalized by the authors and will be added in subsequent PRs. Co-authored-by: @AntoineChambert-Loir --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-number-theory ready-to-merge delegated
label:t-algebra$
373/0 Mathlib.lean,Mathlib/RingTheory/DividedPowers/SubDPIdeal.lean,Mathlib/RingTheory/Ideal/Span.lean 3 20 ['AntoineChambert-Loir', 'github-actions', 'mathlib-bors', 'riccardobrasca'] riccardobrasca
assignee:riccardobrasca
6-35277
6 days ago
6-36888
6 days ago
33-65896
33 days
25235 ADedecker
author:ADedecker
feat: unit space of a (locally) compact T1 monoid is (locally) compact --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-topology 50/0 Mathlib/Topology/Algebra/Constructions.lean,Mathlib/Topology/Algebra/Group/Basic.lean 2 2 ['ADedecker', 'github-actions'] nobody
6-24085
6 days ago
13-30528
13 days ago
13-30513
13 days
25020 erdOne
author:erdOne
feat: define `continuousCohomology` Co-authored-by: Richard Hill --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
244/1 Mathlib.lean,Mathlib/Algebra/Category/ContinuousCohomology/Basic.lean,Mathlib/Algebra/Homology/Embedding/Basic.lean,Mathlib/Algebra/Homology/Embedding/Restriction.lean,Mathlib/CategoryTheory/Limits/Preserves/Shapes/Zero.lean 5 16 ['erdOne', 'github-actions', 'kbuzzard', 'leanprover-community-bot-assistant', 'rmhi'] nobody
6-20226
6 days ago
6-20243
6 days ago
20-22547
20 days
24884 smmercuri
author:smmercuri
feat: `ramificationIdx` for `NumberField.InfinitePlace` --- - [x] depends on: #24880 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-number-theory 38/0 Mathlib/NumberTheory/NumberField/InfinitePlace/Ramification.lean 1 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'riccardobrasca'] nobody
6-19398
6 days ago
21-24116
21 days ago
21-24464
21 days
25119 grunweg
author:grunweg
chore: make `finiteness` a default tactic --- Opening for discussion - [x] depends on: #25111 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author 423/366 Archive/Wiedijk100Theorems/BallotProblem.lean,Mathlib/Analysis/Analytic/Uniqueness.lean,Mathlib/Analysis/Asymptotics/ExpGrowth.lean,Mathlib/Analysis/Calculus/ContDiff/Basic.lean,Mathlib/Analysis/Convex/Integral.lean,Mathlib/Analysis/Fourier/AddCircle.lean,Mathlib/Analysis/Fourier/AddCircleMulti.lean,Mathlib/Analysis/FunctionalSpaces/SobolevInequality.lean,Mathlib/Analysis/Normed/Field/Basic.lean,Mathlib/Analysis/Normed/Lp/PiLp.lean,Mathlib/Analysis/Normed/Lp/ProdLp.lean,Mathlib/Analysis/Normed/Lp/lpSpace.lean,Mathlib/Analysis/SpecialFunctions/Pow/Continuity.lean,Mathlib/Analysis/SpecialFunctions/Pow/NNReal.lean,Mathlib/Analysis/SpecificLimits/Basic.lean,Mathlib/Data/ENNReal/Basic.lean,Mathlib/Data/ENNReal/Holder.lean,Mathlib/Data/ENNReal/Inv.lean,Mathlib/Data/ENNReal/Operations.lean,Mathlib/Data/ENNReal/Real.lean,Mathlib/Data/EReal/Basic.lean,Mathlib/Data/EReal/Operations.lean,Mathlib/InformationTheory/KullbackLeibler/Basic.lean,Mathlib/MeasureTheory/Covering/Besicovitch.lean,Mathlib/MeasureTheory/Function/AEEqOfIntegral.lean,Mathlib/MeasureTheory/Function/ContinuousMapDense.lean,Mathlib/MeasureTheory/Function/ConvergenceInMeasure.lean,Mathlib/MeasureTheory/Function/Egorov.lean,Mathlib/MeasureTheory/Function/Jacobian.lean,Mathlib/MeasureTheory/Function/L1Space/AEEqFun.lean,Mathlib/MeasureTheory/Function/L2Space.lean,Mathlib/MeasureTheory/Function/LocallyIntegrable.lean,Mathlib/MeasureTheory/Function/LpSeminorm/Basic.lean,Mathlib/MeasureTheory/Function/LpSeminorm/ChebyshevMarkov.lean,Mathlib/MeasureTheory/Function/LpSeminorm/CompareExp.lean,Mathlib/MeasureTheory/Function/LpSeminorm/Defs.lean,Mathlib/MeasureTheory/Function/LpSpace/Basic.lean,Mathlib/MeasureTheory/Function/LpSpace/Complete.lean,Mathlib/MeasureTheory/Function/LpSpace/Indicator.lean,Mathlib/MeasureTheory/Function/SimpleFuncDenseLp.lean,Mathlib/MeasureTheory/Function/UniformIntegrable.lean,Mathlib/MeasureTheory/Integral/Bochner/Basic.lean,Mathlib/MeasureTheory/Integral/MeanInequalities.lean,Mathlib/MeasureTheory/Integral/Prod.lean,Mathlib/MeasureTheory/Integral/RieszMarkovKakutani/Real.lean,Mathlib/MeasureTheory/Measure/Decomposition/IntegralRNDeriv.lean,Mathlib/MeasureTheory/Measure/Decomposition/Lebesgue.lean,Mathlib/MeasureTheory/Measure/Haar/Basic.lean,Mathlib/MeasureTheory/Measure/Haar/DistribChar.lean,Mathlib/MeasureTheory/Measure/Haar/Quotient.lean,Mathlib/MeasureTheory/Measure/Haar/Unique.lean,Mathlib/MeasureTheory/Measure/Lebesgue/EqHaar.lean,Mathlib/MeasureTheory/Measure/LevyProkhorovMetric.lean,Mathlib/MeasureTheory/Measure/Real.lean,Mathlib/MeasureTheory/Measure/Restrict.lean,Mathlib/MeasureTheory/Measure/Tilted.lean,Mathlib/MeasureTheory/Measure/Typeclasses/Finite.lean,Mathlib/NumberTheory/NumberField/Discriminant/Basic.lean,Mathlib/Probability/BorelCantelli.lean,Mathlib/Probability/Independence/Conditional.lean,Mathlib/Probability/Integration.lean,Mathlib/Probability/Kernel/Composition/IntegralCompProd.lean,Mathlib/Probability/Kernel/Disintegration/CondCDF.lean,Mathlib/Probability/Kernel/Disintegration/Density.lean,Mathlib/Probability/Martingale/Convergence.lean,Mathlib/Probability/Martingale/OptionalStopping.lean,Mathlib/Probability/Moments/CovarianceBilin.lean,Mathlib/Probability/Moments/Tilted.lean,Mathlib/Probability/Moments/Variance.lean,Mathlib/Probability/UniformOn.lean,Mathlib/Topology/MetricSpace/Bounded.lean,Mathlib/Topology/MetricSpace/Perfect.lean,scripts/noshake.json 73 7 ['github-actions', 'grunweg', 'leanprover-bot', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'sgouezel'] nobody
6-19158
6 days ago
6-31052
6 days ago
6-62051
6 days
22771 alreadydone
author:alreadydone
feat(Homotopy/Lifting): monodromy of a covering map 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 2 ['github-actions', 'mathlib4-dependent-issues-bot'] PatrickMassot
assignee:PatrickMassot
6-18915
6 days ago
82-35471
2 months ago
82-37366
82 days
22279 xyzw12345
author:xyzw12345
feat(RingTheory/GradedAlgebra): homogeneous relation In this PR, we defined the concept of a homogeneous relation and proved some properties about homogeneous relations. The main result of this PR is showing that taking `RingQuot` by a homogeneous relation can give a graded structure on the quotient ring. This result can be used to define graded structures on rings obtained using `RingQuot`, e.g. the Symmetric Algebra defined in #21539 can be verified to have such a structure. Co-authored-by: Zhixuan Dai @atstarrysky <22300180006@m.fudan.edu.cn> Yiming Fu @pelicanhere Zhenyan Fu @pumpkin678 Raphael Douglas Giles @Raph-DG Jiedong Jiang @jjdishere - [x] depends on: #22354 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra
label:t-algebra$
455/0 Mathlib.lean,Mathlib/Algebra/Algebra/Equiv.lean,Mathlib/Algebra/DirectSum/Basic.lean,Mathlib/Algebra/DirectSum/Module.lean,Mathlib/Algebra/Module/LinearMap/Defs.lean,Mathlib/Algebra/RingQuot.lean,Mathlib/RingTheory/GradedAlgebra/Basic.lean,Mathlib/RingTheory/GradedAlgebra/HomogeneousRelation.lean 8 7 ['Paul-Lez', 'github-actions', 'grunweg', 'mathlib4-dependent-issues-bot', 'ocfnash', 'xyzw12345'] ocfnash
assignee:ocfnash
6-18655
6 days ago
68-51515
2 months ago
69-83302
69 days
25406 grunweg
author:grunweg
chore(Linter/DirectoryDependency): move forbidden directories into a JSON file more precisely, to a JSON file with comments: we strip any line beginning with (some whitespace and) the string "// ". Details are up for discussion, such as whether to use toml instead. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-linter 373/306 Mathlib/Tactic/Linter/DirectoryDependency.lean,scripts/README.md,scripts/forbiddenDirs.json 3 2 ['github-actions', 'grunweg'] nobody
6-845
6 days ago
6-7898
6 days ago
6-7949
6 days
22767 robin-carlier
author:robin-carlier
feat(AlgebraicTopology/SimplexCategory): the augmented simplex category This PR defines `AugmentedSimplexCategory` as `WithInitial SimplexCategory`. Using the API in `CategoryTheory.WithTerminal`, we check that functors out of this category (resp. out of its opposite) corresponds to cosimplicial (resp. simplicial) objects, and we link various construction about simplicial objects in terms of this category. --- - [x] depends on : #22658 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory 118/0 Mathlib.lean,Mathlib/AlgebraicTopology/SimplexCategory/Augmented.lean 2 5 ['github-actions', 'joelriou', 'robin-carlier'] joelriou
assignee:joelriou
5-81078
5 days ago
20-23280
20 days ago
90-81566
90 days
22768 robin-carlier
author:robin-carlier
feat(AlgebraicTopology/SimplexCategory/Augmented): monoidal structure on `AugmentedSimplexCategory` We construct a monoidal category structure on `AugmentedSimplexCategory`. The tensor products corresponds to ordinal sum. We characterize morphisms out of a tensor product of object in terms of their precomposition with canonical maps `x ⟶ x ⊗ y` and `y ⟶ x ⊗ y` coming from the fact that the unit is an initial object. Finally, we show that `⦋0⦌` admits a canonical internal monoid object structure. --- - [ ] depends on: #22767 I hope to be able to clear the TODO in `AlgebreaicTopology.SimplexCategory.Augmented.Mon_` in future work, as this should be the "right" statement for the monoidal bar construction, but there is still a long way to go. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory blocked-by-other-PR 560/0 Mathlib.lean,Mathlib/AlgebraicTopology/SimplexCategory/Augmented/Basic.lean,Mathlib/AlgebraicTopology/SimplexCategory/Augmented/Mon_.lean,Mathlib/AlgebraicTopology/SimplexCategory/Augmented/Monoidal.lean,Mathlib/AlgebraicTopology/SimplexCategory/Basic.lean 5 12 ['erdOne', 'github-actions', 'grunweg', 'mathlib4-dependent-issues-bot'] erdOne
assignee:erdOne
5-80608
5 days ago
27-51275
27 days ago
0-33
33 seconds
21969 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 is the first of hopefully many PRs upstreaming work that I have done on diffeological spaces in [my orbifolds repo](https://github.com/peabrainiac/lean-orbifolds), containing the first half of `Diffeology/Basic.lean`. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-differential-geometry 472/0 Mathlib.lean,Mathlib/Geometry/Diffeology/Basic.lean,docs/references.bib,scripts/noshake.json 4 26 ['github-actions', 'grunweg', 'leanprover-community-bot-assistant', 'lecopivo', 'peabrainiac'] fpvandoorn and grunweg
assignee:fpvandoorn assignee:grunweg
5-65792
5 days ago
5-67528
5 days ago
67-59612
67 days
25323 Multramate
author:Multramate
feat(RingTheory/Ideal/Span): add pair lemmas --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
131/31 Mathlib/Algebra/Module/PID.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Affine/Point.lean,Mathlib/RingTheory/DedekindDomain/AdicValuation.lean,Mathlib/RingTheory/Ideal/Maps.lean,Mathlib/RingTheory/Ideal/Span.lean 5 8 ['Multramate', 'eric-wieser', 'github-actions', 'tb65536'] nobody
5-62470
5 days ago
6-76417
6 days ago
6-76401
6 days
24448 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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra awaiting-author
label:t-algebra$
16/1 Mathlib/Algebra/Module/PID.lean,Mathlib/RingTheory/Ideal/Operations.lean,Mathlib/RingTheory/Ideal/Span.lean 3 6 ['Hagb', 'github-actions', 'tb65536'] chrisflav
assignee:chrisflav
5-62465
5 days ago
9-18585
9 days ago
32-8893
32 days
24754 urkud
author:urkud
feat: define `pathIntegral` This is a step towards formalizing of the Poincaré lemma for 1-forms. --- - [x] depends on: #24831 - [x] depends on: #25047 - [x] depends on: #25048 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis awaiting-author 552/8 Mathlib.lean,Mathlib/Analysis/Convex/PathConnected.lean,Mathlib/Analysis/Normed/Module/Basic.lean,Mathlib/MeasureTheory/Integral/IntervalIntegral/Basic.lean,Mathlib/MeasureTheory/Integral/PathIntegral/Basic.lean 5 23 ['github-actions', 'mathlib4-dependent-issues-bot', 'sgouezel', 'urkud'] nobody
5-56092
5 days ago
15-35077
15 days ago
8-52615
8 days
23727 faenuccio
author:faenuccio
chore(RingTheory/Valuation/Discrete/Basic): refactor the definition of discrete valuation to allow for more general targets Co-authored by @mariainesdff The two `ToDo` mentioned in the docstring are WIP by María Inés de Frutos-Fernández and Filippo A. E. Nuccio. --- - [x] depends on: #23725 - [x] depends on: #23726 - [ ] depends on: #24435 large-import t-algebra blocked-by-other-PR WIP
label:t-algebra$
68/26 Mathlib/RingTheory/Valuation/Discrete/Basic.lean 1 31 ['faenuccio', 'github-actions', 'kbuzzard', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'pechersky', 'riccardobrasca'] riccardobrasca
assignee:riccardobrasca
5-46894
5 days ago
5-46896
5 days ago
35-67955
35 days
20238 maemre
author:maemre
feat(Computability/DFA): Closure of regular languages under some set operations This shows that regular languages are closed under complement and intersection by constructing DFAs for them. --- Closure under all other operations will be proved when someone adds the proof for DFA<->regular expression equivalence, so they are not part of this PR. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-zulip t-computability new-contributor awaiting-author 159/0 Mathlib/Computability/DFA.lean,Mathlib/Computability/Language.lean 2 59 ['EtienneC30', 'YaelDillies', 'github-actions', 'maemre', 'meithecatte', 'urkud'] EtienneC30
assignee:EtienneC30
5-43676
5 days ago
34-77815
1 month ago
48-67492
48 days
25236 adomani
author:adomani
feat: the empty line in commands linter This linter flags empty lines within a command. It allows empty lines within doc-strings, module-docs and a couple of other "sensible" places. It also skips files that are likely to contain meta-code, since there the use of empty lines in definition is more widespread. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-linter maintainer-merge 373/11 Archive/Wiedijk100Theorems/BuffonsNeedle.lean,Mathlib.lean,Mathlib/CategoryTheory/Limits/Shapes/NormalMono/Equalizers.lean,Mathlib/Init.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter/EmptyLine.lean,MathlibTest/EmptyLine.lean 7 23 ['adomani', 'bryangingechen', 'github-actions', 'grunweg', 'leanprover-community-bot-assistant'] nobody
5-39042
5 days ago
6-23622
6 days ago
13-20830
13 days
25364 Paul-Lez
author:Paul-Lez
feat(Analysis/SpecialFunction/NthRoot): definition and basic API of Real.nthRoot Co-authored-by: Eric Wieser --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra WIP
label:t-algebra$
256/0 Mathlib/Analysis/SpecialFunctions/NthRoot.lean,Mathlib/Data/Sign.lean 2 16 ['eric-wieser', 'fpvandoorn', 'github-actions', 'j-loreaux', 'madvorak'] nobody
5-35397
5 days ago
7-23524
7 days ago
0-42
42 seconds
24875 smmercuri
author:smmercuri
feat: injectivity of `InfinitePlace.embedding` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-number-theory 19/0 Mathlib/NumberTheory/NumberField/InfinitePlace/Basic.lean 1 6 ['Ruben-VandeVelde', 'github-actions', 'riccardobrasca', 'smmercuri', 'xroblot'] nobody
5-34998
5 days ago
26-48588
26 days ago
26-48642
26 days
25425 Paul-Lez
author:Paul-Lez
feat(LinearAlgebra/Basis/HasCanonicalBasis): propose `HasCanonicalBasis` class Context: in some cases, e.g. writing down PDEs, having a notion of partial derivatives can be useful. In an ideal world (as mentioned by @ocfnash in [this Zulip thread](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Partial.20derivatives/with/463936246)), one could write something along the lines of `open scoped PartialDerivatives` in order to access nice notation for this. This PR introduces a notion of a canonical basis for a module in order to allow taking partial derivatives with respect to it. A later PR (which I am about open) would then propose a notation for taking partial derivatives (defined using `lineDeriv` in order to avoid requiring Frechet-differentiability assumptions). The goal here is to have notation that works equally well on e.g. `𝕜 × 𝕜` and `EuclideanSpace 𝕜 (Fin 2)` and so on. I've opened this PR as a draft in order to get some initial feedback on the content (and whether this is considered appropriate for Mathlib!); the file itself would need to be split (e.g. the instances defined should probably go in different files) Co-authored-by: Eric Wieser --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 105/0 Mathlib.lean,Mathlib/LinearAlgebra/Basis/HasCanonicalBasis.lean 2 1 ['github-actions'] nobody
5-33265
5 days ago
5-37706
5 days ago
0-0
0 seconds
25410 JovanGerb
author:JovanGerb
chore: remove some duplicate instances I have a program that finds duplicate instances, as described at [#mathlib4 > duplicate declarations](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/duplicate.20declarations/with/518941841) This PR is a start at fixing these in Mathlib. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 30/131 Mathlib/Algebra/Category/Grp/Adjunctions.lean,Mathlib/Algebra/Category/ModuleCat/Basic.lean,Mathlib/Algebra/Group/Fin/Basic.lean,Mathlib/Algebra/Homology/Embedding/IsSupported.lean,Mathlib/Algebra/Order/Hom/Monoid.lean,Mathlib/Algebra/Ring/Divisibility/Basic.lean,Mathlib/Algebra/Ring/Subsemiring/Basic.lean,Mathlib/AlgebraicGeometry/Limits.lean,Mathlib/AlgebraicGeometry/OpenImmersion.lean,Mathlib/CategoryTheory/Countable.lean,Mathlib/CategoryTheory/EffectiveEpi/Preserves.lean,Mathlib/CategoryTheory/ObjectProperty/FullSubcategory.lean,Mathlib/Computability/TuringDegree.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/Data/Fintype/EquivFin.lean,Mathlib/Data/List/TakeDrop.lean,Mathlib/Data/Matroid/Constructions.lean,Mathlib/Data/Nat/Basic.lean,Mathlib/Data/Option/Defs.lean,Mathlib/Data/Ordering/Basic.lean,Mathlib/Data/Sign.lean,Mathlib/GroupTheory/Perm/Sign.lean,Mathlib/GroupTheory/Solvable.lean,Mathlib/Logic/Embedding/Basic.lean,Mathlib/Logic/Equiv/Fin/Basic.lean,Mathlib/ModelTheory/Basic.lean,Mathlib/Order/Monotone/Basic.lean,Mathlib/SetTheory/Cardinal/Basic.lean,Mathlib/Tactic/Polyrith.lean,Mathlib/Topology/Compactness/Lindelof.lean 30 9 ['JovanGerb', 'adomani', 'eric-wieser', 'github-actions'] nobody
5-31422
5 days ago
5-77075
5 days ago
5-77059
5 days
21266 ADedecker
author:ADedecker
feat: restate uniformContinuous_mul in terms of convergence to uniformity This is convenient when working with [Filter.Tendsto.congr_uniformity](https://leanprover-community.github.io/mathlib4_docs/Mathlib/Topology/UniformSpace/Basic.html#Filter.Tendsto.congr_uniformity) or [Filter.Tendsto.uniformity_trans](https://leanprover-community.github.io/mathlib4_docs/Mathlib/Topology/UniformSpace/Basic.html#Filter.Tendsto.uniformity_trans), for example. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology easy delegated 8/0 Mathlib/Topology/Algebra/IsUniformGroup/Defs.lean 1 6 ['ADedecker', 'eric-wieser', 'github-actions', 'j-loreaux', 'mathlib-bors'] nobody
5-28956
5 days ago
14-16303
14 days ago
0-18788
5 hours
25429 Paul-Lez
author:Paul-Lez
feat(Analysis/PDE/Quasilinear/Defs): Add definitions about quasilinear first order PDEs This PR introduces some basic definitions related to first order quasilinear PDEs. In a subsequent PR (I'm currently cleaning up the code), these will be used to state and prove some results about how solutions to quasilinear PDEs vary along characteristic curves. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis 141/0 Mathlib.lean,Mathlib/Analysis/PDE/Quasilinear/Defs.lean 2 1 ['github-actions'] nobody
5-25161
5 days ago
5-33331
5 days ago
0-0
0 seconds
25422 xroblot
author:xroblot
feat(NumberField): Image of torsion modulo an ideal Let `I` be an integral ideal of a number field `K`. We define the morphism from the torsion of `K` to `(𝓞 K ⧸ I)ˣ` and prove that it is injective if the norm of `I` is coprime with the order of the torsion of `K`. As a consequence, we prove that for a prime ideal `P` coprime with the order of the torsion of `K`, the norm of `P` is congruent to `1` modulo `torsionOrder K`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-number-theory 202/1 Mathlib.lean,Mathlib/NumberTheory/Cyclotomic/Basic.lean,Mathlib/NumberTheory/Cyclotomic/Rat.lean,Mathlib/NumberTheory/NumberField/Ideal/Basic.lean,Mathlib/RingTheory/RootsOfUnity/PrimitiveRoots.lean 5 1 ['github-actions'] nobody
5-20931
5 days ago
5-21476
5 days ago
5-21470
5 days
25441 kebekus
author:kebekus
feat: introduce the Laplace operator Introduce the Laplace operator for functions on real, finite-dimensional, inner product spaces. 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. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis 197/0 Mathlib.lean,Mathlib/Analysis/Calculus/ContDiff/Basic.lean,Mathlib/Analysis/Calculus/ContDiff/FTaylorSeries.lean,Mathlib/Analysis/InnerProductSpace/Laplace.lean 4 1 ['github-actions'] nobody
5-16852
5 days ago
5-16852
5 days ago
5-16930
5 days
25351 kckennylau
author:kckennylau
feat(CategoryTheory): add API and functoriality for Skeleton --- The `Functor` stuff is really the main content. The `API` stuff is a bit experimental and I don't really know if it's the best approach to do things. I could also make the `API` more functorial, maybe. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-category-theory awaiting-author 51/3 Mathlib/CategoryTheory/Skeletal.lean 1 9 ['github-actions', 'joelriou', 'leanprover-community-bot-assistant'] nobody
5-16373
5 days ago
5-16373
5 days ago
1-39767
1 day
18306 bjoernkjoshanssen
author:bjoernkjoshanssen
feat(Topology/Compactification): projective line over ℝ is homeomorphic to the one-point compactification of ℝ ℙ ℝ (Fin 2 → ℝ) and OnePoint ℝ are homeomorphic: the projective line over ℝ is homeomorphic to the one-point compactification of ℝ. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology awaiting-author 922/0 Mathlib.lean,Mathlib/Topology/Compactification/OnePointHomeomorph.lean,Mathlib/Topology/Compactification/OnePointRealLemmas.lean 3 11 ['bjoernkjoshanssen', 'github-actions', 'leanprover-community-bot-assistant', 'ocfnash'] nobody
5-16176
5 days ago
5-16176
5 days ago
3-38897
3 days
24959 dupuisf
author:dupuisf
feat: the CFC commutes with set integrals This PR shows various versions of `cfc (fun r => ∫ x in s, f x r ∂μ) a = ∫ x in s, cfc (f x) a ∂μ`. We previously had it for integrals over the whole space (i.e. without `s`), but the set version turns out to be very convenient. Lemmas showing the integrability of `fun x => cfc (f x) a` and friends are also added. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-measure-probability t-analysis awaiting-author 377/65 Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Integral.lean 1 23 ['ADedecker', 'dupuisf', 'github-actions', 'j-loreaux'] nobody
5-12489
5 days ago
12-79612
12 days ago
11-4964
11 days
25139 kckennylau
author:kckennylau
feat(RingTheory): basis for `Polynomial.degreeLT` Linear algebra results about the module `R[x]_n` of polynomials with degree `< n`. Co-authored-by: Anne Baanen --- - [x] depends on: #25270 Used in a future resultant PR from branch [kckennylau/resultant](https://github.com/leanprover-community/mathlib4/tree/kckennylau/resultant). This file is split from that branch because there are already over 1000 lines of code. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra awaiting-author
label:t-algebra$
195/2 Mathlib.lean,Mathlib/Algebra/Polynomial/Taylor.lean,Mathlib/RingTheory/Polynomial/DegreeLT.lean 3 108 ['YaelDillies', 'erdOne', 'github-actions', 'kbuzzard', 'kckennylau', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
5-9619
5 days ago
5-43801
5 days ago
4-17234
4 days
20171 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/) new-contributor t-combinatorics awaiting-author 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 18 ['b-mehta', 'github-actions', 'mathlib4-dependent-issues-bot', 'mitchell-horner'] b-mehta
assignee:b-mehta
5-8460
5 days ago
5-18260
5 days ago
21-70934
21 days
25407 adomani
author:adomani
feat: check that the mathlib options exist This PR adds a simple check that all the options mentioned in `mathlibStandardSet` exist (at least, the ones that do exist!). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) maintainer-merge 18/0 Mathlib/Init.lean 1 5 ['adomani', 'github-actions', 'grunweg'] nobody
4-85198
4 days ago
4-85198
4 days ago
5-82859
5 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'] nobody
4-68137
4 days ago
5-6071
5 days ago
6-16421
6 days
23935 Thmoas-Guan
author:Thmoas-Guan
feat(RingTheory/IsSMulRegular): categorical constructions for IsSMulRegular The categorical constructions for `IsSMulRegular` for later use related to `Ext` in a separate file. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-category-theory
label:t-algebra$
62/0 Mathlib.lean,Mathlib/Algebra/Homology/ExactSequence.lean,Mathlib/RingTheory/Regular/Category.lean 3 36 ['Thmoas-Guan', 'erdOne', 'github-actions', 'joelriou', 'riccardobrasca'] joelriou
assignee:joelriou
4-54006
4 days ago
17-33074
17 days ago
49-76048
49 days
25259 Thmoas-Guan
author:Thmoas-Guan
feat(Algebra): associated primes of localized module We proved the `Ass(S^{-1}M)` is equal to the preimage of `Ass(M)` under `Ideal.comap` when over noetherian ring. From this we proved that every minimal primes 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$
70/11 Mathlib/RingTheory/Ideal/AssociatedPrime/Localization.lean 1 6 ['Thmoas-Guan', 'erdOne', 'github-actions', 'leanprover-community-bot-assistant'] nobody
4-53977
4 days ago
11-30057
11 days ago
12-23956
12 days
25213 mbkybky
author:mbkybky
feat(RingTheory/KrullDimension): Krull Dimension of quotient regular sequence We show that if `M` is a finite module over a Noetherian local ring `R`, `[r₁, …, rₙ]` is an `M`-sequence, then `dim M⧸(r₁, …, rₙ)M + n = dim M`. Co-authored-by: Nailin Guan @Thmoas-Guan - [x] depends on: #24771 - [x] depends on: #25210 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
241/24 Mathlib.lean,Mathlib/Algebra/Module/Submodule/Lattice.lean,Mathlib/LinearAlgebra/Quotient/Basic.lean,Mathlib/RingTheory/Ideal/MinimalPrime/Localization.lean,Mathlib/RingTheory/KrullDimension/Module.lean,Mathlib/RingTheory/KrullDimension/Regular.lean,Mathlib/RingTheory/Nakayama.lean,Mathlib/RingTheory/Spectrum/Prime/LTSeries.lean,Mathlib/RingTheory/Support.lean 9 n/a ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
4-53955
4 days ago
unknown
unknown
24249 Thmoas-Guan
author:Thmoas-Guan
feat(Algebra): the Rees theorem for depth In this PR we proved the Rees theorem for depth. Co-authored-by: Hu Yongle --- - [ ] depends on: #23937 - [ ] depends on: #24244 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-algebra blocked-by-other-PR
label:t-algebra$
370/2 Mathlib.lean,Mathlib/Algebra/Category/Grp/Preadditive.lean,Mathlib/Algebra/Homology/ExactSequence.lean,Mathlib/RingTheory/Regular/Category.lean,Mathlib/RingTheory/Regular/Depth.lean 5 n/a ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
4-53839
4 days ago
unknown
unknown
24246 Thmoas-Guan
author:Thmoas-Guan
feat(Algebra): Ext iso quotient regular sequence In this PR defined the `addequiv` between `Ext M N k` and `N =>[R] M/ rs * M` where `rs` is a regular sequence of length `k` Co-authored-by: Hu Yongle Co-authored-by: Wang Jingting --- - [ ] depends on: #23937 - [ ] depends on: #24244 - [ ] depends on: #24249 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-algebra blocked-by-other-PR
label:t-algebra$
430/2 Mathlib.lean,Mathlib/Algebra/Category/Grp/Preadditive.lean,Mathlib/Algebra/Homology/ExactSequence.lean,Mathlib/RingTheory/Regular/Category.lean,Mathlib/RingTheory/Regular/Depth.lean 5 n/a ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
4-53794
4 days ago
unknown
unknown
23937 Thmoas-Guan
author:Thmoas-Guan
feat(Algebra): vanishing of induced hom between ext In this PR we proved that the induced map `Ext(N,M)` -> `Ext(N,M)` from the left scalar multiple on `M` with `x` when `x` in `ann(N)` is zero. Co-authored-by: Wang Jingting Co-authored-by: Hu Yongle --- - [x] depends on: #19591 - [x] depends on: #23690 - [ ] depends on: #23935 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-category-theory blocked-by-other-PR WIP
label:t-algebra$
148/0 Mathlib.lean,Mathlib/Algebra/Homology/ExactSequence.lean,Mathlib/RingTheory/Regular/Category.lean 3 n/a ['Thmoas-Guan', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
4-53780
4 days ago
unknown
unknown
24921 Thmoas-Guan
author:Thmoas-Guan
feat(Algebra): definition of depth In this PR, we defined the depth of two modules as the minimal order of nonvanishing `Ext` and the `I-depth` for ideal `I` and some basic properties. Including the equivalence of the two in the condition of rees theorem. --- - [ ] depends on: #24249 - [ ] depends on: #24244 - [ ] depends on: #23937 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-algebra blocked-by-other-PR
label:t-algebra$
663/2 Mathlib.lean,Mathlib/Algebra/Category/Grp/Preadditive.lean,Mathlib/Algebra/Homology/ExactSequence.lean,Mathlib/RingTheory/Regular/Category.lean,Mathlib/RingTheory/Regular/Depth.lean 5 n/a ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
4-53766
4 days ago
unknown
unknown
24923 Thmoas-Guan
author:Thmoas-Guan
feat(Algebra): Auslander-Buchsbaum theorem This PR mainly proved the Auslander-Buchsbaum theorem stating for a noetherian local ring `R` and a finitely generated `R` module `M` , `proj.dim(M) + depth(M) = depth(R)`. Co-authored-by: Yongle Hu --- - [ ] depends on: #24921 - [ ] depends on: #24249 - [x] depends on: #24734 - [x] depends on: #24697 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-algebra blocked-by-other-PR
label:t-algebra$
1188/2 Mathlib.lean,Mathlib/Algebra/Category/Grp/Preadditive.lean,Mathlib/Algebra/Homology/ExactSequence.lean,Mathlib/RingTheory/Regular/AuslanderBuchsbaum.lean,Mathlib/RingTheory/Regular/Category.lean,Mathlib/RingTheory/Regular/Depth.lean 6 n/a ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
4-53707
4 days ago
unknown
unknown
25109 Thmoas-Guan
author:Thmoas-Guan
feat(Algebra): depth of QuotSMulTop In this PR, we proved for a local ring `R` and a finitely generated `R` module `M N`, `IsSMulRegular M x` and `x ∈ Module.annihilator R N`, then `depth(N, M/xM) + 1 = depth(N, M)`, and its corollary for quotient regular seqence. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-algebra
label:t-algebra$
949/2 Mathlib.lean,Mathlib/Algebra/Category/Grp/Preadditive.lean,Mathlib/Algebra/Homology/ExactSequence.lean,Mathlib/RingTheory/Regular/Category.lean,Mathlib/RingTheory/Regular/Depth.lean 5 n/a ['github-actions'] nobody
4-53662
4 days ago
unknown
unknown
24922 Thmoas-Guan
author:Thmoas-Guan
feat(Algebra): Ischebeck theorem This PR mainly proved the Ischbecke theorem, stating that `depth(N,M)` is greater or equal to `depth(M) - dim(N)` for finitely generated module `N, M` over local ring. --- - [ ] depends on: #24921 - [ ] depends on: #24249 - [ ] depends on: #24771 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-algebra blocked-by-other-PR WIP
label:t-algebra$
1020/2 Mathlib.lean,Mathlib/Algebra/Category/Grp/Preadditive.lean,Mathlib/Algebra/Homology/ExactSequence.lean,Mathlib/RingTheory/Regular/Category.lean,Mathlib/RingTheory/Regular/Depth.lean,Mathlib/RingTheory/Regular/Ischebeck.lean 6 n/a ['Thmoas-Guan', 'github-actions', 'mathlib4-dependent-issues-bot'] nobody
4-53613
4 days ago
unknown
unknown
25223 kckennylau
author:kckennylau
feat(Algebra): Quadratic Algebra --- WIP. Please adopt. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra please-adopt WIP
label:t-algebra$
153/0 Mathlib.lean,Mathlib/Algebra/QuadraticAlgebra.lean 2 3 ['github-actions', 'mans0954'] nobody
4-47922
4 days ago
13-76292
13 days ago
0-31
31 seconds
25287 digama0
author:digama0
feat(Bicategory/CatEnriched): 2-cat from Cat-enriched cat A construction of the canonical strict bicategory structure given a `EnrichedCategory Cat C`. From the ∞-cosmos project. Co-Authored-By: Emily Riehl --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) infinity-cosmos t-category-theory awaiting-author 129/0 Mathlib.lean,Mathlib/CategoryTheory/Bicategory/CatEnriched.lean 2 17 ['digama0', 'emilyriehl', 'github-actions', 'joelriou', 'peabrainiac', 'yuma-mizuno'] nobody
4-45264
4 days ago
4-45264
4 days ago
7-22660
7 days
25347 sgouezel
author:sgouezel
feat: define Riemannian manifolds We introduce typeclasses to deal with Riemannian manifolds: * In a fiber bundle whose fibers are already endowed with an inner product space structure, `[IsContinuousRiemannianBundle F E]` registers the fact the inner product depends continuously on the base point. This is a Prop-valued class, on top of existing data `[∀ x, NormedAddCommGroup (E x)]` `[∀ x, InnerProductSpace ℝ (E x)]`. * We also register `[IsContMDiffRiemannianBundle n IB F E]` similarly. * There is an issue when the fibers already have a topological structure (for instance the tangent spaces), because adding an assumption `[∀ x, NormedAddCommGroup (TangentSpace I x)]` would create a diamond. Instead, we introduce another typeclass `[RiemannianBundle E]` containing the data of an inner product space on the fibers, compatible with the preexisting topology. From this class, we register instances of inner product space structures on the fibers, whose topology is defeq to the original one. * We make sure that registering concrete instances of `[RiemannianBundle E]` registers automatically `[IsContinuousRiemannianBundle F E]` and/or `[IsContMDiffRiemannianBundle n IB F E]` in terms of the regularity of the metric. * Under the assumptions `[RiemannianBundle (fun (b : M) -> TangentSpace I b)]` and `[EMetricSpace M]`, we register a Prop-valued typeclass `[IsRiemannianManifold I M]` registering the fact that the edist coincides with the infimum of the lengths of paths, measured using the normed space structure in the tangent spaces. With this design, one can develop the general theory of Riemannian bundles and Riemannian manifolds, and also define concrete instances. When working with a generic Riemannian manifold, the typeclasses will include (in addition to the usual one for manifolds, replacing the topological space one with an emetric space one) the assumptions `[RiemannianBundle (fun (b : M) -> TangentSpace I b)]` `[IsContinuousRiemannianBundle E (fun (b : M) -> TangentSpace I b)]` `[IsContMDiffRiemannianBundle n I E (fun (b : M) -> TangentSpace I b)]`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-differential-geometry WIP 981/56 Mathlib.lean,Mathlib/Analysis/Normed/Operator/BoundedLinearMaps.lean,Mathlib/Analysis/NormedSpace/OperatorNorm/NormedSpace.lean,Mathlib/Data/Bundle.lean,Mathlib/Geometry/Manifold/ContMDiff/NormedSpace.lean,Mathlib/Geometry/Manifold/Riemannian/Basic.lean,Mathlib/Geometry/Manifold/VectorBundle/Basic.lean,Mathlib/Geometry/Manifold/VectorBundle/Hom.lean,Mathlib/Geometry/Manifold/VectorBundle/Riemannian.lean,Mathlib/Geometry/Manifold/VectorBundle/Tangent.lean,Mathlib/Topology/FiberBundle/Basic.lean,Mathlib/Topology/FiberBundle/Constructions.lean,Mathlib/Topology/FiberBundle/Trivialization.lean,Mathlib/Topology/Homeomorph/Defs.lean,Mathlib/Topology/VectorBundle/Basic.lean,Mathlib/Topology/VectorBundle/Constructions.lean,Mathlib/Topology/VectorBundle/Hom.lean,Mathlib/Topology/VectorBundle/Riemannian.lean 18 4 ['github-actions', 'leanprover-bot', 'sgouezel'] nobody
4-41422
4 days ago
4-43956
4 days ago
0-1
1 second
25474 adomani
author:adomani
test for .lean/.md check A test PR for #25473. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) file-removed 10/1 .github/workflows/lint_and_suggest_pr.yml,Mathlib.lean,Mathlib/NumberTheory/NumberField/CMField.Lean 3 1 ['github-actions'] nobody
4-36516
4 days ago
4-37849
4 days ago
4-37907
4 days
24769 YaelDillies
author:YaelDillies
feat: `X ⟶ M` is a commutative monoid if `M` is a commutative monoid object Also add a shortcut `Grp_.homMk` of `Mon_.Hom.mk` for `Grp_`, provide Yoneda-like lemmas for monoid morphisms and bundle `Mon_.ext` into an `Injective` lemma. Unsimp `Grp_Class.tensorHom_inv_inv_mul` since it loops with `IsMon_Hom.mul_hom` + `IsMon_Hom ι`. 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-category-theory 73/10 Mathlib/CategoryTheory/Monoidal/Cartesian/Grp_.lean,Mathlib/CategoryTheory/Monoidal/Cartesian/Mon_.lean,Mathlib/CategoryTheory/Monoidal/Grp_.lean,Mathlib/CategoryTheory/Monoidal/Mon_.lean 4 35 ['YaelDillies', 'erdOne', 'github-actions', 'joelriou', 'leanprover-community-bot-assistant', 'robin-carlier'] nobody
4-35619
4 days ago
4-35679
4 days ago
28-30332
28 days
11968 JovanGerb
author:JovanGerb
feat: improvements to RefinedDiscrTree This PR defines `RefinedDiscrTree`, which is an improved version of `DiscrTree` with many new features, such as - indexing lambda terms, dependent forall terms, and bound variables. - giving a score to matches, in order to sort them - indexing star patterns so that `a+b` and `a+a` are indexed differently - taking into account eta reductions, so that `exp` can still be matched with the library pattern `fun x => exp (f x)`. This PR makes `RefinedDiscrTree` into a lazy data structure, meaning that it can be used without a cache, just like `LazyDiscrTree`. This PR also removes these features: - indexing `fun x => x` as `id` - indexing `fun x => f x + g x` as `f + g`, and similarly for `-`, `*`, `/`, `⁻¹`, `^`. - indexing `fun _ => 42` as `42` These equivalent indexings do not hold definitionally in the `reducible` transparency, which is the transparency that is used for unification when using a discrimination tree. Therefore, indexing these different expressions the same is actually inefficient rather than helpful. This is part of the bigger #11768, which uses this discrimination tree for a library rewriting tactic. This replaces an older version of `RefinedDiscrTree`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) file-removed new-contributor t-meta 1631/1242 Mathlib.lean,Mathlib/Lean/Meta/RefinedDiscrTree.lean,Mathlib/Lean/Meta/RefinedDiscrTree/Basic.lean,Mathlib/Lean/Meta/RefinedDiscrTree/Encode.lean,Mathlib/Lean/Meta/RefinedDiscrTree/Initialize.lean,Mathlib/Lean/Meta/RefinedDiscrTree/Lookup.lean,Mathlib/Lean/Meta/RefinedDiscrTree/Pi.lean,Mathlib/Tactic.lean,Mathlib/Tactic/FunProp.lean,Mathlib/Tactic/FunProp/Elab.lean,Mathlib/Tactic/FunProp/StateList.lean,Mathlib/Tactic/FunProp/Theorems.lean,Mathlib/Tactic/FunProp/Types.lean,Mathlib/Topology/Defs/Basic.lean,MathlibTest/RefinedDiscrTree.lean,scripts/noshake.json 16 79 ['0art0', 'JovanGerb', 'eric-wieser', 'github-actions', 'grunweg', 'joneugster', 'leanprover-bot', 'leanprover-community-bot-assistant', 'rosborn'] nobody
4-35094
4 days ago
4-85032
4 days ago
237-83175
237 days
25453 JovanGerb
author:JovanGerb
perf(Algebra/Homology/HomotopyCategory): use explicit universe parameter in `Category` As we have seen before, writing `Category.{v}` instead of `Category` avoids a nasty universe level metavariable, and this helps to speed up unification. The changes in this PR are somewhat arbitrary, but it serves as an example for this principle. --- [![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'] nobody
4-32725
4 days ago
5-373
5 days ago
5-427
5 days
24465 adomani
author:adomani
feat: a linter to enforce formatting This linter enforces that the hypotheses of every declaration are correctly formatted. This already required multiple PRs to make mathlib compliant. Ideally, little by little the linter can be extended to format more of mathlib. --- The default linter option is `false`, but the lakefile enforces it to be `true`. This means that the linter does not run on `MathlibTest`. However, the tests should still be compliant, since the default option was `true` in development and the tests were fixed. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-linter maintainer-merge 876/4 Mathlib.lean,Mathlib/Algebra/Group/Int/Defs.lean,Mathlib/Algebra/Group/Nat/Defs.lean,Mathlib/Algebra/Ring/Int/Defs.lean,Mathlib/Data/FunLike/Basic.lean,Mathlib/Data/SetLike/Basic.lean,Mathlib/Init.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter/CommandStart.lean,Mathlib/Tactic/Simps/NotationClass.lean,MathlibTest/CommandStart.lean,MathlibTest/EuclideanSpace.lean,MathlibTest/Simps.lean,MathlibTest/Traversable.lean,MathlibTest/antidiagonal.lean,MathlibTest/delabLinearIndependent.lean,MathlibTest/matrix.lean,MathlibTest/norm_num.lean,MathlibTest/set_like.lean,MathlibTest/vec_notation.lean 20 89 ['Parcly-Taxel', 'adomani', 'eric-wieser', 'github-actions', 'grunweg', 'leanprover-community-bot-assistant'] grunweg
assignee:grunweg
4-30689
4 days ago
27-42382
27 days ago*
40-47103
40 days*
25473 adomani
author:adomani
feat(CI): check that Mathlib files have lean or md extension Twice recently there have been files with an "intended" `.lean` extension in `Mathlib/`: * #24942, ending in `;lean`; * #25457, ending in `.Lean`. `mk_all` does not add these files to `Mathlib.lean`, since they do not end in `.lean` and this later causes problems. This CI step checks that all files in `Mathlib/` end with `.lean` or `.md`. See #25474 for a test where the new step [correctly fails](https://github.com/leanprover-community/mathlib4/actions/runs/15464097783/job/43532018379?pr=25474). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) CI delegated 10/0 .github/workflows/lint_and_suggest_pr.yml 1 10 ['adomani', 'bryangingechen', 'github-actions', 'grunweg', 'mathlib-bors'] nobody
4-25952
4 days ago
4-26842
4 days ago
0-11212
3 hours
25482 grunweg
author:grunweg
chore(aesop_cat): update comment Since mathlib includes leanprover/lean4#7448, update the comment accordingly. #25475 shows that this fast-path is still beneficial: so leave it, but update its comment accordingly. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory 4/4 Mathlib/CategoryTheory/Category/Basic.lean 1 2 ['JovanGerb', 'github-actions', 'grunweg'] nobody
4-24173
4 days ago
4-26873
4 days ago
4-26925
4 days
25484 VTrelat
author:VTrelat
feat(SetTheory/ZFC/Booleans): define Boolean algebra in ZFC Extend the model of ZFC with Boolean algebra: - define a set 𝔹 of booleans - define a proper type `ZFBool` representing booleans - add theorems on usual algebraic properties of booleans - provide usual boolean notations like `⊤`, `⊥`, `∧`, `∨`, etc. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) - [ ] depends on: #25483 new-contributor blocked-by-other-PR 619/0 Mathlib/Data/Set/Prod.lean,Mathlib/SetTheory/ZFC/Basic.lean,Mathlib/SetTheory/ZFC/Booleans.lean 3 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
4-24128
4 days ago
4-24130
4 days ago
0-1523
25 minutes
25485 VTrelat
author:VTrelat
feat(SetTheory/ZFC/Naturals): define natural numbers in ZFC Extend the model of ZFC with naturals: - define a set `Nat` of naturals following the usual construction (∅, {∅}, {∅, {∅}}, ...) - define a proper type `ZFNat` representing naturals - add theorems on usual algebraic properties of naturals - provide a recursor and induction schemes to define/prove by induction --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) - [ ] depend on: #25483 new-contributor 2095/0 Mathlib/Data/Set/Prod.lean,Mathlib/SetTheory/ZFC/Basic.lean,Mathlib/SetTheory/ZFC/Booleans.lean,Mathlib/SetTheory/ZFC/Naturals.lean 4 1 ['github-actions'] nobody
4-22216
4 days ago
4-22281
4 days ago
4-22277
4 days
25265 FMLJohn
author:FMLJohn
feat(Order/SupClosed): `compl_image_latticeClosure` and `compl_image_latticeClosure_eq_of_compl_image_eq_self` The main results in this pull request are: 1. `compl_image_latticeClosure`: given any Boolean algebra `α` and `s : Set α`, `compl '' latticeClosure s` is the same as `latticeClosure (compl '' s)`; 2. `compl_image_latticeClosure_eq_of_compl_image_eq_self`: given any Boolean algebra `α` and `s : Set α` such that `compl '' s = s`, we have `compl '' latticeClosure s = latticeClosure s`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) maintainer-merge t-order 59/1 Mathlib/Order/SupClosed.lean 1 8 ['FMLJohn', 'YaelDillies', 'github-actions'] bryangingechen
assignee:bryangingechen
4-22149
4 days ago
7-2121
7 days ago
11-11741
11 days
25369 Paul-Lez
author:Paul-Lez
feat(Order/Fin/CircularOrder): add some basic results about the circular order on Fin Co-authored-by: Oliver Nash --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order awaiting-author 33/0 Mathlib.lean,Mathlib/Order/Circular.lean,Mathlib/Order/Fin/CircularOrder.lean 3 11 ['Paul-Lez', 'YaelDillies', 'eric-wieser', 'github-actions'] bryangingechen
assignee:bryangingechen
4-22121
4 days ago
4-22121
4 days ago
2-19068
2 days
25483 VTrelat
author:VTrelat
chore(Data/Set/Prod, SetTheory/ZFC/Basic): add theorem prod_subset_of_prod and extend ZFC model Required by @eric-wieser in #24281 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data new-contributor 103/0 Mathlib/Data/Set/Prod.lean,Mathlib/SetTheory/ZFC/Basic.lean 2 2 ['VTrelat', 'github-actions'] nobody
4-20161
4 days ago
4-26780
4 days ago
4-26834
4 days
25488 VTrelat
author:VTrelat
feat(SetTheory/ZFC/Rationals): define rationals in ZFC Extend the model of ZFC with rationals: we define a proper type `ZFRat` representing integers based on pairs of `ZFInt` (enforcing the res to be nonzero) and following the usual construction of rationals. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) - [ ] depends on: #25483 - [ ] depends on: #25485 - [ ] depends on: #25486 new-contributor blocked-by-other-PR 2070/0 Mathlib/Data/Set/Prod.lean,Mathlib/SetTheory/ZFC/Basic.lean,Mathlib/SetTheory/ZFC/Booleans.lean,Mathlib/SetTheory/ZFC/Integers.lean,Mathlib/SetTheory/ZFC/Rationals.lean 5 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
4-19805
4 days ago
4-19807
4 days ago
0-1808
30 minutes
25486 VTrelat
author:VTrelat
feat(SetTheory/ZFC/Integers): define integers in ZFC Extend the model of ZFC with integers following the converse direction as for naturals. We first define a type and then build a set. We finally show that both representations have coercions in both direction: - define a proper type `ZFInt` representing integers based on `ZFNat × ZFNat` and following the usual construction of integers - add theorems on usual algebraic properties of integers - define a set `Int` and show that it matches-i.e. that it is isomorphic to-the type `ZFInt` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) - [ ] depends on: #25483 - [ ] depends on: #25485 new-contributor blocked-by-other-PR 2003/0 Mathlib/Data/Set/Prod.lean,Mathlib/SetTheory/ZFC/Basic.lean,Mathlib/SetTheory/ZFC/Booleans.lean,Mathlib/SetTheory/ZFC/Integers.lean 4 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
4-19803
4 days ago
4-19805
4 days ago
0-2067
34 minutes
24321 peabrainiac
author:peabrainiac
feat(CategoryTheory/Adjunction): more results on adjoint triples. Lemmas about adjoint triples `F ⊣ G ⊣ H` where either `G` is fully faithful or `F` and `H` are. From [lean-orbifolds](https://github.com/peabrainiac/lean-orbifolds/blob/387fe778f3cc1ed3c5e60f390842333ecc9eda67/Orbifolds/ForMathlib/Triple.lean). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory awaiting-author 255/19 Mathlib/CategoryTheory/Adjunction/Triple.lean,Mathlib/CategoryTheory/EpiMono.lean 2 14 ['github-actions', 'joelriou', 'leanprover-bot', 'peabrainiac'] nobody
4-17509
4 days ago
4-17509
4 days ago
22-20077
22 days
25493 IvanRenison
author:IvanRenison
feat(Analysis/InnerProductSpace/Positive): add theorem `IsPositive.nonneg_eigenvalues` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-analysis 8/0 Mathlib/Analysis/InnerProductSpace/Positive.lean 1 1 ['github-actions'] nobody
4-16988
4 days ago
4-16994
4 days ago
4-17054
4 days
25172 eric-wieser
author:eric-wieser
feat: restricting `Affine.Simplex` to an affine subspace that contains it Also removes a redundant `Nonempty` argument. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) maintainer-merge t-euclidean-geometry 68/5 Mathlib/LinearAlgebra/AffineSpace/AffineSubspace/Basic.lean,Mathlib/LinearAlgebra/AffineSpace/Independent.lean 2 10 ['eric-wieser', 'github-actions', 'jsm28', 'ocfnash'] nobody
4-16192
4 days ago
15-26171
15 days ago
15-67045
15 days
25254 fpvandoorn
author:fpvandoorn
fix: cleanup measurability + prod/sum lemmas + fun_prop * Add `fun_prop` to a few more lemmas * Rename the compositional version to something without a prime, add the compositional version for `StronglyMeasurable` * use the `prod/fun_prod` naming scheme (the compositional version is called `prod_apply`) for `[AE][Strongly]Measurable` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-measure-probability awaiting-author 128/50 Mathlib/MeasureTheory/Function/StronglyMeasurable/AEStronglyMeasurable.lean,Mathlib/MeasureTheory/Function/StronglyMeasurable/Basic.lean,Mathlib/MeasureTheory/Function/UniformIntegrable.lean,Mathlib/MeasureTheory/Group/Arithmetic.lean,Mathlib/Probability/Integration.lean,Mathlib/Probability/Martingale/Basic.lean,Mathlib/Probability/Martingale/BorelCantelli.lean,Mathlib/Probability/Martingale/Centering.lean 8 6 ['fpvandoorn', 'github-actions', 'sgouezel'] nobody
4-12035
4 days ago
4-22296
4 days ago
1-38112
1 day
25427 Paul-Lez
author:Paul-Lez
feat(Analysis/Calculus/PartialDerivatives): Propose notation for partial derivatives. This PR introduces a notation for partial derivatives, taken with respect to a canonical basis. The idea here is that this might be useful for e.g. writing down PDEs. The notation allows use to write things like ```lean -- The canonical basis for `ℝ × ℝ` is indexed by `Fin 0` so `∂₀[ℝ]` corresponds to taking -- the first partial derivative example : (∂₀[ℝ] fun (x : ℝ × ℝ) => x.1) 0 = 1 := by simp [Pi.zero_def, lineDeriv] ``` This has already been discussed on Zulip [here](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Partial.20derivatives). I've opened this PR as a draft in order to get preliminary feedback on the contents (e.g. is this appropriate for Mathlib?); the file contains some demos of the notation in action. Co-authored-by: Eric Wieser --- - [ ] depends on: #25425 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR 195/0 Mathlib.lean,Mathlib/Analysis/Calculus/PartialDerivatives/Notation.lean,Mathlib/LinearAlgebra/Basis/HasCanonicalBasis.lean 3 13 ['github-actions', 'lecopivo', 'mathlib4-dependent-issues-bot', 'ocfnash'] nobody
4-9860
4 days ago
5-34143
5 days ago
0-0
0 seconds
23413 robin-carlier
author:robin-carlier
feat(CategoryTheory/Join): Pseudofunctoriality of joins of categories Promote the constructions `C ↦ C ⋆ D` and `D ↦ C ⋆ D` to pseudofunctors from `Cat` to `Cat`. The construction is carried in a new file `CategoryTheory/Join/Pseudofunctor.lean` to reduce imports. --- - [x] depends on: #23412 The pseudofunctoriality statements here are not the most general. The "right" statements would be 1) "pseudobifunctoriality". 2) pseudofunctoriality with values in slice bicategories. Unfortunately, the two-categorical machinery in mathlib is not advanced enough yet to even make sense of the statements (first would require at least product bicategories, or 2-categories of pseudofunctors for a curried version, second would require slice bicategories.). The content of this file should be upgraded once said constructions in bicategories are available, but for now I want at least to have statements that recover what we already have for `WithInitial` and `WithTerminal` rather than conditioning everything on a (probably rather long) bicategorical sidequest. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory 169/0 Mathlib.lean,Mathlib/CategoryTheory/Join/Basic.lean,Mathlib/CategoryTheory/Join/Pseudofunctor.lean 3 10 ['github-actions', 'joelriou', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'robin-carlier'] nobody
4-202
4 days ago
4-224
4 days ago
51-19980
51 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 78/3 Mathlib/Util/Delaborators.lean,Mathlib/Util/PPOptions.lean,MathlibTest/delaborators.lean 3 1 ['github-actions'] nobody
3-83296
3 days ago
3-83304
3 days ago
3-83365
3 days
25255 Raph-DG
author:Raph-DG
feat(RingTheory): Order of vanishing in a ring In this PR we define the order of vanishing of a ring and its extension to elements of the function field (as in stacks project 02MD) as well as some basic API. Note that I'm slightly unsure that some of the lemmas used to prove this are at the right level of generality, and further I'm not quite sure where some of these lemmas belong (as indicated by the comments in the main OrderOfVanishing.lean file). Any comments about this would be very much appreciated. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) maintainer-merge new-contributor t-algebra RFC
label:t-algebra$
247/0 Mathlib.lean,Mathlib/Algebra/Order/Monoid/Unbundled/WithTop.lean,Mathlib/RingTheory/Artinian/Module.lean,Mathlib/RingTheory/Ideal/Operations.lean,Mathlib/RingTheory/Ideal/Quotient/Operations.lean,Mathlib/RingTheory/OrderOfVanishing.lean 6 83 ['Raph-DG', 'chrisflav', 'erdOne', 'github-actions', 'jcommelin'] nobody
3-81423
3 days ago
3-82009
3 days ago
10-61393
10 days
25218 kckennylau
author:kckennylau
feat(AlgebraicGeometry): Tate normal form of elliptic curves --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-zulip new-contributor t-algebraic-geometry 291/26 Mathlib.lean,Mathlib/AlgebraicGeometry/EllipticCurve/IsomOfJ.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Modular/TateNormalForm.lean,Mathlib/AlgebraicGeometry/EllipticCurve/NormalForms.lean,Mathlib/AlgebraicGeometry/EllipticCurve/VariableChange.lean 5 29 ['MichaelStollBayreuth', 'Multramate', 'acmepjz', 'github-actions', 'grunweg', 'kckennylau'] nobody
3-79757
3 days ago
7-32169
7 days ago
6-51040
6 days
22137 grunweg
author:grunweg
feat: `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 will be used in my bordism theory project. ------------ - [x] depends on: #22827 (for breaking the import cycle) - [ ] depends on: #25510 (shuffling homeomorphism properties around, to avoid a non-linear dependency - [x] depends on: #22969 - [x] depends on: #22964 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-topology awaiting-author blocked-by-other-PR 196/71 Mathlib/Data/Sum/Basic.lean,Mathlib/Topology/Constructions/SumProd.lean 2 23 ['github-actions', 'grunweg', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'plp127'] nobody
3-60871
3 days ago
3-60873
3 days ago
0-0
0 seconds
25510 grunweg
author:grunweg
chore(Topology/Constructions/SumProd.lean): split homeomorphism properties section Move properties about products to the products section, and sum properties to the sum section: this is necessary for #22137, which will use homeomorphism properties for sums for inducing maps. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology 81/71 Mathlib/Topology/Constructions/SumProd.lean 1 1 ['github-actions'] nobody
3-60375
3 days ago
3-61728
3 days ago
3-61714
3 days
24669 qawbecrdtey
author:qawbecrdtey
feat(Analysis/Normed/Operator/LinearIsometry): added definition `LinearIsometryEquiv.prodComm` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) This commit defines a `LinearIsometryEquiv`, and states some trivial theorems about it. ```lean def prodComm [Module R E₂] : E × E₂ ≃ₗᵢ[R] E₂ × E ``` maintainer-merge t-analysis 21/1 Mathlib/Analysis/Normed/Operator/LinearIsometry.lean 1 7 ['Ruben-VandeVelde', 'eric-wieser', 'faenuccio', 'github-actions', 'jcommelin', 'qawbecrdtey'] faenuccio
assignee:faenuccio
3-57041
3 days ago
5-39681
5 days ago
32-56510
32 days
25450 pechersky
author:pechersky
feat(Valued): Valuation.leAddSubgroup and ideal/submodule versions of ltAddSubgroup Also prove that these are clopen. Factored out of #24627 Fix capitalization spelling mistake on `closedball` in a lemma --- [![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$
272/30 Mathlib/RingTheory/Valuation/Basic.lean,Mathlib/RingTheory/Valuation/Integers.lean,Mathlib/Topology/Algebra/Valued/LocallyCompact.lean,Mathlib/Topology/Algebra/Valued/ValuationTopology.lean 4 4 ['faenuccio', 'github-actions', 'pechersky'] nobody
3-56323
3 days ago
5-5847
5 days ago
5-7366
5 days
24627 pechersky
author:pechersky
feat(Topology/Algebra/Valued): `IsLinearTopology 𝒪[K] K` and `𝒪[K] 𝒪[K]` as well as `IsLinearTopology ℤ_[p] ℤ_[p]` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) - [ ] depends on: #25450 t-topology awaiting-author blocked-by-other-PR 376/30 Mathlib.lean,Mathlib/NumberTheory/Padics/LinearTopology.lean,Mathlib/RingTheory/Valuation/Basic.lean,Mathlib/RingTheory/Valuation/Integers.lean,Mathlib/Topology/Algebra/Valued/LinearTopology.lean,Mathlib/Topology/Algebra/Valued/LocallyCompact.lean,Mathlib/Topology/Algebra/Valued/ValuationTopology.lean,Mathlib/Topology/Algebra/Valued/ValuedField.lean 8 40 ['ADedecker', 'faenuccio', 'github-actions', 'loefflerd', 'mathlib4-dependent-issues-bot', 'pechersky'] nobody
3-55509
3 days ago
5-5130
5 days ago
19-50489
19 days
23669 erdOne
author:erdOne
feat(FieldTheory): abelian extensions --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra awaiting-author
label:t-algebra$
74/0 Mathlib.lean,Mathlib/FieldTheory/Galois/Abelian.lean,Mathlib/NumberTheory/Cyclotomic/Gal.lean 3 6 ['acmepjz', 'alreadydone', 'chrisflav', 'erdOne', 'github-actions', 'xroblot'] nobody
3-50620
3 days ago
36-34663
1 month ago
29-68817
29 days
25522 grunweg
author:grunweg
chore: add ContinuousLinearEquiv.prodAssoc A continuous version of LinearEquiv.prodAssoc. Part of #25505 (on the path towards defining submanifolds). --- - [ ] depends on: #23971 for simplicity [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR 127/30 Mathlib/Analysis/Convolution.lean,Mathlib/Analysis/NormedSpace/OperatorNorm/Prod.lean,Mathlib/LinearAlgebra/Prod.lean,Mathlib/NumberTheory/NumberField/CanonicalEmbedding/Basic.lean,Mathlib/Topology/Algebra/Module/Equiv.lean,Mathlib/Topology/VectorBundle/Constructions.lean 6 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
3-47026
3 days ago
3-47028
3 days ago
0-568
9 minutes
25505 grunweg
author:grunweg
feat: a `SliceModel` typeclass for models with corners for embedded submanifolds TODO: write a proper PR description (once things settle down a bit, and the dependent PRs have landed) Then ask e.g. Sebastien for review. Rebased and extended version of #24550: - on the current master branch - does not import the definition of smooth immersions/embeddings: this only defines slice models (no more) --- - [ ] depends on: #23971 - [ ] depends on: #25522 - [ ] depends on: #25524 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-differential-geometry blocked-by-other-PR WIP 288/0 Mathlib.lean,Mathlib/Geometry/Manifold/SliceModel.lean 2 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
3-44397
3 days ago
3-59499
3 days ago
0-2
2 seconds
21265 ADedecker
author:ADedecker
feat: some lemmas about pointwise actions of units on filters and uniformities --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-topology delegated
label:t-algebra$
45/0 Mathlib/Order/Filter/Pointwise.lean,Mathlib/Topology/Algebra/UniformMulAction.lean 2 8 ['github-actions', 'grunweg', 'mathlib-bors', 'ocfnash'] nobody
3-43644
3 days ago
114-83977
3 months ago
15-25642
15 days
22366 kim-em
author:kim-em
feat: `check_equalities` tactic for diagnosing defeq problems The `check_equalities` tactic, which checks the typing of equalities in the goal, reporting discrepancies between the implicit type argument of the equality, and the inferred types of the left and right hand sides, at "instances and reducible" transparency. Reports from this tactic do not necessarily indicate a problem, although typically `simp` should reduce rather than increase the reported discrepancies. `check_equalities` may be useful in diagnosing uses of `erw`. t-meta delegated 119/3 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Basic.lean,Mathlib/Tactic/CategoryTheory/CheckCompositions.lean,Mathlib/Tactic/CheckEqualities.lean,Mathlib/Tactic/Common.lean,MathlibTest/check_equalities.lean 7 13 ['adomani', 'b-mehta', 'eric-wieser', 'github-actions', 'grunweg', 'mathlib-bors'] nobody
3-43553
3 days ago
87-17765
2 months ago
15-14325
15 days
18693 Ruben-VandeVelde
author:Ruben-VandeVelde
feat: add ConjRootClass Co-authored-by: FR --- From #6718 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra delegated
label:t-algebra$
213/0 Mathlib.lean,Mathlib/FieldTheory/Minpoly/ConjRootClass.lean,Mathlib/FieldTheory/Minpoly/IsConjRoot.lean 3 16 ['LessnessRandomness', 'Vierkantor', 'alreadydone', 'github-actions', 'grunweg', 'mathlib-bors'] Vierkantor
assignee:Vierkantor
3-43512
3 days ago
14-19065
14 days ago
94-8480
94 days
25326 YaelDillies
author:YaelDillies
feat: `Mon_ C` is cartesian-monoidal if `C` is From Toric --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) toric t-category-theory 36/0 Mathlib/CategoryTheory/Monoidal/Cartesian/Basic.lean,Mathlib/CategoryTheory/Monoidal/Cartesian/Mon_.lean 2 3 ['github-actions', 'joelriou', 'leanprover-community-bot-assistant'] nobody
3-43510
3 days ago
3-43579
3 days ago
8-7875
8 days
23971 grunweg
author:grunweg
feat: ContinuousLinearEquiv.{prodUnique,uniqueProd} which are `LinearEquiv.{prodUnique,uniqueProd}` as a continuous linear equivalence. Discovered when working on slice models for defining submanifolds (#24550), one step towards defining smooth submanifolds. --- - [x] depends on: #24168 (for the LinearEquiv) part - [x] depends on: #25513 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
61/3 Mathlib/LinearAlgebra/Prod.lean,Mathlib/Topology/Algebra/Module/Equiv.lean 2 9 ['Ruben-VandeVelde', 'github-actions', 'grunweg', 'j-loreaux', 'mathlib4-dependent-issues-bot'] nobody
3-37622
3 days ago
3-38594
3 days ago
10-52636
10 days
23674 xroblot
author:xroblot
feat(NumberField/IsCM): first results about the action of `complexConjugation` on units --- - [x] depends on: #23536 - [x] depends on: #23453 - [ ] depends on: #23684 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-number-theory blocked-by-other-PR 227/72 Mathlib/Algebra/Field/Equiv.lean,Mathlib/Algebra/Group/Invertible/Basic.lean,Mathlib/AlgebraicGeometry/Morphisms/Proper.lean,Mathlib/FieldTheory/LinearDisjoint.lean,Mathlib/GroupTheory/GroupAction/FixedPoints.lean,Mathlib/LinearAlgebra/Dimension/Localization.lean,Mathlib/NumberTheory/NumberField/CMField.lean,Mathlib/NumberTheory/NumberField/Units/Basic.lean,Mathlib/RingTheory/Artinian/Ring.lean,Mathlib/RingTheory/IntegralClosure/Algebra/Defs.lean,Mathlib/RingTheory/IntegralClosure/IsIntegralClosure/Basic.lean,Mathlib/RingTheory/LinearDisjoint.lean,Mathlib/RingTheory/Localization/FractionRing.lean,Mathlib/RingTheory/Localization/Integral.lean,Mathlib/RingTheory/SimpleRing/Field.lean 15 4 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
3-37572
3 days ago
3-37580
3 days ago
0-703
11 minutes
23992 robertmaxton42
author:robertmaxton42
feat (Limits.FunctorCategory): limitIsoFlipCompLim and colimitIsoFlipCompColim are natural Add `limIsoFlipCompWhiskerLim`, `limCompFlipIsoWhiskerLim`, `colimIsoFlipCompWhiskerColim`, `colimCompFlipIsoWhiskerColim`, each witnessing that their corresponding families of isomorphisms are natural in the diagram $F$. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-category-theory awaiting-CI 41/0 Mathlib/CategoryTheory/Limits/FunctorCategory/Basic.lean 1 12 ['adomani', 'github-actions', 'robertmaxton42', 'robin-carlier'] nobody
3-34653
3 days ago
3-76008
3 days ago
50-83251
50 days
24593 Multramate
author:Multramate
refactor(AlgebraicGeometry/EllipticCurve/*): replace Fin 3 with products This allows the removal of all instances of `erw` in `Jacobian` and `Projective` files. --- - [x] depends on: #21356 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebraic-geometry 1000/1022 Mathlib/AlgebraicGeometry/EllipticCurve/Jacobian/Basic.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Jacobian/Formula.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Jacobian/Point.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Projective/Basic.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Projective/Formula.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Projective/Point.lean 6 n/a ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
3-34471
3 days ago
unknown
unknown
25030 Multramate
author:Multramate
feat(NumberTheory/EllipticDivisibilitySequence): add elliptic nets Defines elliptic nets and redefines elliptic sequences using elliptic relators. This is part of #13057 by Junyan Xu. Co-authored-by: Junyan Xu --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-number-theory 259/37 Mathlib/NumberTheory/EllipticDivisibilitySequence.lean 1 1 ['github-actions'] nobody
3-33209
3 days ago
17-77730
17 days ago
17-77714
17 days
25132 Multramate
author:Multramate
chore(NumberTheory/EllipticDivisibilitySequence): rename definitions --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-number-theory WIP 265/45 Mathlib/NumberTheory/EllipticDivisibilitySequence.lean 1 2 ['github-actions', 'leanprover-community-bot-assistant'] nobody
3-33201
3 days ago
3-33894
3 days ago
0-1
1 second
25524 grunweg
author:grunweg
feat: EuclideanSpace.finAddEquivProd I need this for #25505 (to show that R^n is a submanifold of R^m for n \leq m) and for my bordism theory branch. Previous zulip discussions: - [#Is there code for X? > Product of Euclidean spaces @ 💬](https://leanprover.zulipchat.com/#narrow/channel/217875-Is-there-code-for-X.3F/topic/Product.20of.20Euclidean.20spaces/near/500124944) - [#mathlib4 > Create `LinearIsometryEquiv` with `WithLp 2 (α × β)` and.. @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Create.20.60LinearIsometryEquiv.60.20with.20.60WithLp.202.20.28.CE.B1.20.C3.97.20.CE.B2.29.60.20and.2E.2E/near/505938119) - [#mathlib4 > Manifold structure on Moebius strip @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Manifold.20structure.20on.20Moebius.20strip/near/522156122) Co-authored-by: @peabrainiac --- TODO: paste my zulip reasoning above into the PR description. I still believe my applications 1 and 2 may hold water, but 3/4 may not. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis 21/0 Mathlib/Analysis/InnerProductSpace/PiL2.lean 1 5 ['eric-wieser', 'github-actions', 'grunweg'] nobody
3-29993
3 days ago
3-45111
3 days ago
3-45170
3 days
22611 grunweg
author:grunweg
feat: disjoint unions distribute with products of manifolds Prove an analogue of [Equiv.prodSumDistrib](https://leanprover-community.github.io/mathlib4_docs/Mathlib/Logic/Equiv/Basic.html#Equiv.prodSumDistrib) and [Homeomorph.prodSumDistrib](https://leanprover-community.github.io/mathlib4_docs/Mathlib/Topology/Homeomorph.html#Homeomorph.prodSumDistrib) for smooth manifolds: disjoint unions and products of manifolds are distributive, up to canonical diffeomorphism. This is (up to lots of abstraction) the key result for proving distributivity of the bordism ring. This proof depends on two sorries: - if a function has bijective `mfderiv` at `x`, it is a local diffeomorphism at `x`. This follows from the inverse function theorem for manifolds; I have an old branch which needs *just* a little more work. - injectivity of the differential of the respective map; this will follow from basic API about `mfderiv` for products and disjoint unions (which is currently missing); I will add that anyway Labelling as please-adopt as help with both of these is welcome. I'll be happy to share my progress towards the two sorries. --- - [x] depends on: #23969 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-differential-geometry please-adopt WIP 75/6 Mathlib/Geometry/Manifold/Diffeomorph.lean,Mathlib/Geometry/Manifold/LocalDiffeomorph.lean 2 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
3-29903
3 days ago
3-30839
3 days ago
0-0
0 seconds
24917 adomani
author:adomani
feat: deprecated module automation This PR is a revised version of #24861. It splits the `#create_deprecated_modules` into two commands: * `#create_deprecated_module path/to/file.lean` that guides you through generating a deprecated file; * `#find_deleted_files n` that looks at the repository `n` commits ago and returns a `#create_deprecated_module` for each file that existed then and does not exist now. This is integrated with `Try these:` suggestions and is intended as a first step in making this process completely automatic. Each regenerated file consists of just the imports of the last file that existed, before deletion, followed by `deprecated_import (since := "YYYY-MM-DD")`. In particular, this also applies to *renames*, where it might be more natural to suggest the renamed file, rather than its imports. However, this is part of the deprecation logic that I consider best left to a possible future PR, since distinguishing renames from removals is a separate matter that even git does not handle completely satisfactorily. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta awaiting-author 374/0 scripts/README.md,scripts/create_deprecated_modules.lean 2 42 ['YaelDillies', 'adomani', 'github-actions', 'grunweg'] grunweg
assignee:grunweg
3-28364
3 days ago
3-28364
3 days ago
21-26659
21 days
25529 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 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology 229/1 Counterexamples.lean,Counterexamples/TopologistsSineCurve.lean,Mathlib/Topology/Connected/PathConnected.lean 3 4 ['github-actions', 'grunweg', 'loefflerd'] nobody
3-27952
3 days ago
3-39699
3 days ago
3-39753
3 days
24441 MrSumato
author:MrSumato
feat(Data/List): add Lyndon-Schutzenberger theorem on list commutativity Add Lyndon-Schutzenberger theorem on list commutativity. Included definition for List.repeatSelf that returns list repeated n times. --- This is my first mathlib PR, so any comments are highly appreciated. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data new-contributor awaiting-author 129/1 Mathlib.lean,Mathlib/Data/List/Commutativity.lean,Mathlib/Data/List/Defs.lean,Mathlib/Data/List/Lemmas.lean 4 35 ['MrSumato', 'github-actions', 'grunweg', 'plp127'] grunweg
assignee:grunweg
3-25453
3 days ago
3-25453
3 days ago
29-59355
29 days
25025 scholzhannah
author:scholzhannah
feat(Topology/CWComplex/Classical/Basic.lean): basic lemmas about CW complexes This PR has a few basic lemmas about (classical) CW complexes that will be necessary for the addition of subcomplexes. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology awaiting-author 44/2 Mathlib/Topology/CWComplex/Classical/Basic.lean 1 5 ['github-actions', 'grunweg'] grunweg
assignee:grunweg
3-24876
3 days ago
3-24876
3 days ago
17-72261
17 days
25362 adomani
author:adomani
feat: a linter for duplicated `open` This linter warns when a namespace is repeated. It makes an effort to report only the problematic namespaces, but is not especially robust. The linter has some awareness of the `namespace` command, so ```lean def X.Y := 0 open X namespace X open Y ``` will flag both `namespace X` and `open Y` as problematic, even though it was the `open `X` that became redundant with `namespace X`. However, I will not have much time to devote to polishing this and there are quite a few exception in Mathlib before a better version could be seriously considered for adoption. [#mathlib4 > linter requests @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/linter.20requests/near/520273644) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import please-adopt 177/28 Mathlib.lean,Mathlib/Data/Fin/Basic.lean,Mathlib/Init.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Bound.lean,Mathlib/Tactic/Linarith/Oracle/FourierMotzkin.lean,Mathlib/Tactic/Linter.lean,Mathlib/Tactic/Linter/DupOpen.lean,Mathlib/Tactic/NormNum/PowMod.lean,Mathlib/Tactic/ReduceModChar.lean,Mathlib/Tactic/Widget/StringDiagram.lean,Mathlib/Topology/CWComplex/Abstract/Basic.lean,Mathlib/Topology/ContinuousMap/Interval.lean,Mathlib/Topology/Germ.lean,Mathlib/Topology/Homotopy/HSpaces.lean,Mathlib/Topology/Order/LowerUpperTopology.lean,Mathlib/Topology/Order/PartialSups.lean,Mathlib/Topology/Separation/DisjointCover.lean,Mathlib/Topology/Sheaves/Sheafify.lean,MathlibTest/DupOpen.lean 20 13 ['adomani', 'github-actions', 'grunweg', 'leanprover-community-bot-assistant'] nobody
3-23334
3 days ago
6-12843
6 days ago
0-0
0 seconds
25516 kim-em
author:kim-em
chore: test PR from fork This PR tests making a PR from a fork. 1/0 Mathlib/Computability/AkraBazzi/AkraBazzi.lean 1 1 ['bryangingechen'] nobody
3-22035
3 days ago
3-58538
3 days ago
0-0
0 seconds
23240 urkud
author:urkud
feat(Topology/Maps): `IsOpenMap` and `ClusterPt` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology delegated 17/4 Mathlib/Topology/Maps/Basic.lean 1 8 ['eric-wieser', 'github-actions', 'grunweg', 'mathlib-bors', 'urkud'] nobody
3-20874
3 days ago
77-76255
2 months ago
0-12104
3 hours
25537 literandltx
author:literandltx
feat(number_theory/legendre_symbol): Add sqrt‐of‐residue theorems for p=4k+3 and p=8k+5 Add a new file `QuadraticResidueRoots.lean` under `Mathlib/NumberTheory/LegendreSymbol/` that proves two explicit “square-root of quadratic residue” theorems for primes of the specific form. - **`exists_sqrt_of_residue_mod4_eq3`** for primes `p = 4*k + 3` - **`exists_sqrt_of_residue_mod8_eq5`** for primes `p = 8*k + 5` It also introduces the helper lemmas `euler_criterion_traditional` and `legendreSym.at_two_mod8_eq_5`. Import lines in `Mathlib.lean` and `Mathlib/NumberTheory/LegendreSymbol/Basic.lean` have been updated accordingly. new-contributor 217/0 Mathlib.lean,Mathlib/NumberTheory/LegendreSymbol/Basic.lean,Mathlib/NumberTheory/LegendreSymbol/QuadraticReciprocity.lean,Mathlib/NumberTheory/LegendreSymbol/QuadraticResidueRoots.lean 4 0 [] nobody
3-19735
3 days ago
3-19735
3 days ago
0-0
0 seconds
25318 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. Co-authored-by: Floris van Doorn --- - [ ] depends on: #21237 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology 175/5 Mathlib/Topology/Compactness/CompactlyCoherentSpace.lean 1 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
3-16736
3 days ago
3-26961
3 days ago
5-20518
5 days
8167 sebzim4500
author:sebzim4500
feat: a `grw` tactic for rewriting using inequalities Co-authored-by: @hrmacbeth, @digama0 --- - [x] depends on: #8796 ```lean example (x y z w : ℝ) (h₁ : x < z) (h₂ : w ≤ y + 4) (h₃ : Real.exp z < 5 * w) : Real.exp x < 5 * (y + 4) := by grw [h₁, ← h₂] exact h₃ ``` [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-meta modifies-tactic-syntax awaiting-author 552/2 Mathlib.lean,Mathlib/Data/Int/ModEq.lean,Mathlib/Tactic.lean,Mathlib/Tactic/GCongr/Core.lean,Mathlib/Tactic/GRW.lean,Mathlib/Tactic/GRW/Core.lean,Mathlib/Tactic/GRW/Lemmas.lean,MathlibTest/GRW.lean,scripts/noshake.json 9 61 ['JLimperg', 'JovanGerb', 'Vierkantor', 'digama0', 'eric-wieser', 'fpvandoorn', 'github-actions', 'hrmacbeth', 'kim-em', 'leanprover-community-mathlib4-bot', 'sebzim4500'] nobody
3-2362
3 days ago
12-11127
12 days ago
111-42249
111 days
25499 robin-carlier
author:robin-carlier
feat(CategoryTheory/Monoidal): left action of monoidal categories Define (left) actions of a monoidal category on a category: a `MonoidalLeftAction` of a monoidal category `C` on a category `D` consists of an action bifunctor `- ⊙ - : C ⥤ D ⥤ D`, equipped with structural natural isomorphisms `(- ⊗ -) ⊙ - ≅ - ⊙ - ⊙ -` and `𝟙_ C ⊙ - ≅ -`, subject to coherence conditions. The code in this PR is parallel to the existing code for monoidal category. We provide a battery of basic `simp` lemmas to ease working with this type class, and show that every monoidal category acts on itself via its tensor product. The code is put in a new subdirectory `CategoryTheory/Monoidal/Action`. Future wok on the subject includes - Providing a constructor for `MonoidalLeftAction` taking a monoidal functor from `C` to `D ⥤ D`, where the latter has the "composition" monoidal structure. - Constructing the action of `C ⥤ C` on `C`. - Extending the notion of module objects internal to a monoidal category to allow the `Mon_ ` object to be in `C`, and the module to be in `D` where `D` has a monoidal left action of `C`. - Using the two previous points, show that given a monad `M`, there is an equivalence of categories between `Algebra M` and modules in `C` over the monoid `M.toMon : Mon_ (C ⥤ C)̀`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory 348/0 Mathlib.lean,Mathlib/CategoryTheory/Monoidal/Action/Basic.lean,docs/references.bib 3 1 ['github-actions'] nobody
3-429
3 days ago
3-12085
3 days ago
3-85883
3 days
25545 robin-carlier
author:robin-carlier
refactor(CategoryTheory/Monoidal/Mod_): refactor `Mod_` using `MonoidalLeftAction` Generalize the definition of `CategoryTheory.Monoidal.Mod_Class` and `CategoryTheory.Monoidal.Mod_` to modules in `D` over a monoid object in `C`, where `C` acts monoidally on `D`. At the same time, we refactor `Mod_` in a way similar to the one `Mon_` has been refactored in #24646. i.e we favor `Mod_Class` in the definition and `Mod_`, and introduce a Prop-class `IsMod_Hom` to define morphisms of modules. --- - [ ] depends on: #25499 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory blocked-by-other-PR 551/112 Mathlib.lean,Mathlib/CategoryTheory/Monoidal/Action/Basic.lean,Mathlib/CategoryTheory/Monoidal/Cartesian/Mod_.lean,Mathlib/CategoryTheory/Monoidal/Mod_.lean,docs/references.bib 5 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
2-86281
2 days ago
3-424
3 days ago
0-459
7 minutes
22586 joelriou
author:joelriou
feat(CategoryTheory/Localization): the right derivability structure given by functorial resolutions In this PR, we provide a constructor for right derivability structures. We assume that `Φ : LocalizerMorphism W₁ W₂` is given by a fully faithful functor `Φ.functor : C₁ ⥤ C₂` and that we have a resolution functor `ρ : C₂ ⥤ C₁` with a natural transformation `i : 𝟭 C₂ ⟶ ρ ⋙ Φ.functor` such that `W₂ (i.app X₂)` for any `X₂ : C₂`. If we assume that `W₁` is induced by `W₂`, that `W₂` is multiplicative and has the two out of three property, then `Φ` is a right derivability structure. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory 153/0 Mathlib.lean,Mathlib/CategoryTheory/Localization/DerivabilityStructure/OfFunctorialResolutions.lean,Mathlib/CategoryTheory/Localization/LocalizerMorphism.lean 3 13 ['github-actions', 'joelriou', 'robin-carlier'] nobody
2-83814
2 days ago
2-83814
2 days ago
92-80070
92 days
24612 Paul-Lez
author:Paul-Lez
feat(Tactic/ImportDiff): add `#import_diff` command This PR adds the `#import_diff` command, which lists new transitive imports added by extending the list of imports of a file. The aim of this command is to help with debugging large import changes. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) will-close-soon t-meta awaiting-author 35/0 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/ImportDiff.lean 3 8 ['adomani', 'github-actions', 'joneugster'] adomani and joneugster
assignee:joneugster assignee:adomani
2-82314
2 days ago
2-82314
2 days ago
2-61262
2 days
25548 robin-carlier
author:robin-carlier
chore(CategoryTheory/Limits/Shape/End): define coends The content of `CategoryTheory/Limits/Shapes/End` was not dualized, so only ends where defined, but not coends. This PR dualizes the content of the file: we introduce `Cowedge`s as special kinds of `Multicofork`s, and define the `coend_ F` as the colimit of a canonical cowedge we can build from `F : Jᵒᵖ ⥤ J ⥤ C`. Also, we rename `CategoryTheory.Limits.hom_ext` to `CategoryTheory.Limits.end_.hom_ext`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory 137/7 Mathlib/CategoryTheory/Limits/Shapes/End.lean,Mathlib/CategoryTheory/Limits/Shapes/Multiequalizer.lean 2 1 ['github-actions'] nobody
2-79904
2 days ago
2-79904
2 days ago
2-79943
2 days
24540 robertmaxton42
author:robertmaxton42
feat(Quiv): add the empty, vertex, point, interval, and walking quivers Add: * The empty quiver * The vertex quiver (one vertex, and no edges) and the point quiver (one vertex, one self-edge) * The interval quiver (two vertices with an edge between them) * The walking quiver (vertices `0` and `1` with two edges both `0 -> 1`. Functors from the walking quiver to `Type` define quivers, by interpreting `F.obj 0` as the type of vertices, `F.obj 1` as the type of edges, using one of the two edges to label the source of every edge and using the other to label the target.) - [x] depends on: #24538 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory awaiting-author 370/0 Mathlib.lean,Mathlib/CategoryTheory/Category/Quiv/Shapes.lean,Mathlib/CategoryTheory/Category/Quiv/WalkingQuiver.lean,Mathlib/Logic/Small/Defs.lean 4 12 ['github-actions', 'joelriou', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'robertmaxton42', 'robin-carlier'] nobody
2-76295
2 days ago
2-76295
2 days ago
0-80193
22 hours
25550 eric-wieser
author:eric-wieser
doc: explain the fields of MonadWriter --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data documentation 11/3 Mathlib/Control/Monad/Writer.lean 1 1 ['github-actions'] nobody
2-75463
2 days ago
2-75463
2 days ago
2-77548
2 days
25534 JovanGerb
author:JovanGerb
feat: let `gcongr` deal with implications This PR implements support for the `_ → _` relation in the `gcongr` tactic. This can be useful in its own right, but the main reason for this is to later implement the `grw` and `gconvert` tactic using this infrastructure. To be more specific, `_ → _` is now supported as a relation, *and* as a constant. Supporting it as a constant is not necessary for the purpose of `grw`, but it seems natural to add support for it in this PR, so that lemmas like `imp_imp_imp` can be used by `gcongr`. To make `_ → _` in `gcongr` work more easily out of the box, I've built in support for goals of the form `r a b → r c d` where `r` is a transitive relation (i.e. it implements `isTrans α r`). This behaviour can be overridden with a `@[gcongr]` tag, and this is in particular done for the `<` relation, since we want the new goals to use `≤` instead of `<`. [#mathlib4 > Rewrite with inequalities @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Rewrite.20with.20inequalities/near/522751787) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-meta 280/93 Mathlib/Tactic/Core.lean,Mathlib/Tactic/GCongr.lean,Mathlib/Tactic/GCongr/Core.lean,Mathlib/Tactic/GCongr/CoreAttrs.lean,MathlibTest/GCongr/implications.lean,MathlibTest/GCongr/inequalities.lean,MathlibTest/GCongr/mod.lean,scripts/noshake.json 8 6 ['JovanGerb', 'github-actions', 'grunweg'] nobody
2-74970
2 days ago
2-75464
2 days ago
3-19120
3 days
25556 Parcly-Taxel
author:Parcly-Taxel
chore: remove >6 month old material in `Deprecated` file-removed tech debt 0/250 Mathlib.lean,Mathlib/Deprecated/Cardinal/Continuum.lean,Mathlib/Deprecated/Cardinal/Finite.lean,Mathlib/Deprecated/Cardinal/PartENat.lean,Mathlib/Deprecated/Order.lean 5 1 ['github-actions'] nobody
2-55793
2 days ago
2-55846
2 days ago
2-55905
2 days
25459 emilyriehl
author:emilyriehl
Feat(CategoryTheory): terminal categories with an application to hoFunctor Some preliminary API around terminal categories is developed with an application for the infinity-cosmos project: proving that the homotopy category functor preserves terminal objects. We also include proofs that `[0]` is terminal in the simplex category and `Δ[0]` is the terminal simplicial set. Co-authored by [Robin Carlier](robin.carlier@ens-lyon.fr), [Adam Topaz](topaz@ualberta.ca), and [Zeyi Zhao](zzhao95@jh.edu). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) infinity-cosmos large-import t-category-theory 178/3 Mathlib.lean,Mathlib/AlgebraicTopology/SimplexCategory/Basic.lean,Mathlib/AlgebraicTopology/SimplicialSet/HomotopyCat.lean,Mathlib/AlgebraicTopology/SimplicialSet/Monoidal.lean,Mathlib/CategoryTheory/Category/Cat/Terminal.lean,Mathlib/CategoryTheory/Category/ReflQuiv.lean,Mathlib/CategoryTheory/Quotient.lean 7 3 ['emilyriehl', 'github-actions', 'jcommelin'] nobody
2-47711
2 days ago
4-23991
4 days ago
4-81274
4 days
19860 YaelDillies
author:YaelDillies
refactor: review the `simps` projections of `OneHom`, `MulHom`, `MonoidHom` Make `simps` generate `coe_concreteHom` rather than`concreteHom_apply`. From FLT --- In fact, I would love to have both the `coe_` and `_apply` projections simultaneously and also to not have to specify ` simps (config := .asFn))` every single time we want to generate the `coe_` projection, but `simps ` seems to not be able to do that? cc @fpvandoorn I must say, after four years of working on mathlib, I still don't understand how one is supposed to use `simps`. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra awaiting-CI
label:t-algebra$
100/118 Mathlib/Algebra/BigOperators/Group/Multiset/Basic.lean,Mathlib/Algebra/Group/Hom/Defs.lean,Mathlib/Algebra/Group/Subgroup/Defs.lean,Mathlib/Algebra/Group/Submonoid/Operations.lean,Mathlib/Algebra/Group/WithOne/Basic.lean,Mathlib/Algebra/GroupWithZero/WithZero.lean,Mathlib/Algebra/Module/End.lean,Mathlib/GroupTheory/NoncommCoprod.lean 8 4 ['fpvandoorn', 'github-actions', 'leanprover-community-bot-assistant'] nobody
2-41818
2 days ago
2-41839
2 days ago
0-17
17 seconds
25215 mans0954
author:mans0954
feature(RingTheory/RootsOfUnity/Basic) : rootsOfUnity coercions For a commutative monoid, `rootsOfUnity` can be coerced to the set `{z : R | z^k = 1}`. For a commutative ring which is a domain, `rootsOfUnity` can be coerced to `nthRootsFinset k (1 : R)`. Zulip discussion: https://leanprover.zulipchat.com/#narrow/channel/116395-maths/topic/roots.20of.20unity.20-.20computing.20low.20degree/with/520362922 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
22/0 Mathlib/RingTheory/RootsOfUnity/Basic.lean 1 1 ['github-actions'] nobody
2-39154
2 days ago
14-10564
14 days ago
14-10619
14 days
24828 mans0954
author:mans0954
feature(Algebra/Polynomial/Roots) : nthRoots_two_unit_of_char_ne_two Compute the second roots of the unit for rings of characteristic not 2. See also: #25215 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
11/0 Mathlib/Algebra/Polynomial/Roots.lean,Mathlib/Data/Multiset/ZeroCons.lean 2 1 ['github-actions'] nobody
2-39084
2 days ago
27-53731
27 days ago
27-59865
27 days
25175 zcyemi
author:zcyemi
feat(Geometry/Euclidean/Congurence): add triangle congruence Add triangle congruence theorems. --- Some parts of the [original PR](https://github.com/leanprover-community/mathlib3/pull/18214) in Lean 3 have already been migrated to mathlib4: `Mathlib.Topology.MetricSpace.Congruence` and `Mathlib.Topology.MetricSpace.Similarity`. Therefore, I just rearranged the file and left the core triangle congruence proofs here. I'm not sure whether we need a standalone `Congruence.lean` file or if we should merge these into `Triangle.lean`. The law of sines was commited with another PR. Discussion on [zulip](https://leanprover.zulipchat.com/#narrow/channel/217875-Is-there-code-for-X.3F/topic/Law.20of.20Sines.20for.20Euclidean.20Geometry.20Triangles/near/520245156) - [ ] depends on: #25174 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-euclidean-geometry blocked-by-other-PR 211/1 Mathlib/Geometry/Euclidean/Congruence.lean,Mathlib/Geometry/Euclidean/Triangle.lean 2 12 ['JovanGerb', 'github-actions', 'mathlib4-dependent-issues-bot'] nobody
2-38945
2 days ago
15-47839
15 days ago
0-1224
20 minutes
21026 joelriou
author:joelriou
feat(CategoryTheory/Limits): certain multicoequalizers are pushouts In this file, we show that a multicoequalizer for for `I : MultispanIndex (.ofLinearOrder ι) C` is also a pushout when `ι` has exactly two elements. --- - [x] depends on: #22203 - [x] depends on: #20988 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory 81/0 Mathlib.lean,Mathlib/CategoryTheory/Limits/Shapes/MultiequalizerPullback.lean 2 13 ['erdOne', 'github-actions', 'joelriou', 'mathlib4-dependent-issues-bot', 'robin-carlier'] nobody
2-37313
2 days ago
2-39279
2 days ago
42-7640
42 days
25557 AntoineChambert-Loir
author:AntoineChambert-Loir
feat(Data.Nat.LogFueled): fueled version of `clog` This is an attempt to `fuel` docs#Nat.clog (and similar functions, later on, with the intent of making docs#primeFactorsList being computed). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data WIP 201/0 Mathlib.lean,Mathlib/Data/Nat/LogFueled.lean 2 1 ['github-actions'] nobody
2-36506
2 days ago
2-44998
2 days ago
0-60
1 minute
25059 s235282
author:s235282
feat(Combinatorics/SimpleGraph/Bipartite): a graph is 2-colorable iff it's bipartite Define a predicate for a simple graph to be bipartite (`def IsBipartite (G : SimpleGraph V) : Prop := G.Colorable 2`) and prove ` G.IsBipartite ↔ ∃ s t : Set V, G.IsBipartiteWith s t`. --- This is my first attempt at contributing to mathlib and therefore I have a couple of points of uncertainty related to: - Naming conventions for theorems - Seeing a lot of isBipartite vs IsBipartite in the original work. What do we want to go with when? - Definition placement - Where should I put the IsBipartite definition. - Structure of biimplication theorems - Should I combine the different lemmas into 1 bgi theorem? Feedback is greatly appreciated :) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import maintainer-merge new-contributor t-combinatorics 36/3 Mathlib/Combinatorics/SimpleGraph/Bipartite.lean 1 30 ['YaelDillies', 'github-actions', 'mitchell-horner', 's235282'] nobody
2-36455
2 days ago
2-37002
2 days ago
8-84432
8 days
24261 Paul-Lez
author:Paul-Lez
chore: replace `WithLp.equiv` with a new pair `WithLp.toLp`/`WithLp.ofLp` This PR does the following: - deprecate `WithLp.equiv` - Add `WithLp.toLp` and `WithLp.ofLp` (for consistency with other equivalences to type synonyms) See [Zulip discussion](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/defeq.20abuse.20in.20.60WithLp.60) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis 759/366 Mathlib/Algebra/Module/ZLattice/Covolume.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/Matrix.lean,Mathlib/Analysis/Normed/Algebra/UnitizationL1.lean,Mathlib/Analysis/Normed/Lp/PiLp.lean,Mathlib/Analysis/Normed/Lp/ProdLp.lean,Mathlib/Analysis/Normed/Lp/WithLp.lean,Mathlib/Analysis/Quaternion.lean,Mathlib/Analysis/RCLike/Inner.lean,Mathlib/Analysis/SpecialFunctions/Gaussian/FourierTransform.lean,Mathlib/Combinatorics/Additive/AP/Three/Behrend.lean,Mathlib/Geometry/Euclidean/Angle/Unoriented/CrossProduct.lean,Mathlib/LinearAlgebra/Matrix/Hermitian.lean,Mathlib/LinearAlgebra/Matrix/LDL.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,MathlibTest/EuclideanSpace.lean 24 50 ['Paul-Lez', 'YaelDillies', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant'] nobody
2-35204
2 days ago
2-35224
2 days ago
33-31560
33 days
24661 edegeltje
author:edegeltje
feat(Tactic/Algebraize): Allow the `algebraize` tactic to use lemmas which don't (directly) mention RingHom This PR allows the `algebraize` tactic to be applied in more cases. Specifically, in cases where the assumption is not (directly) about RingHom, it should still be able to apply lemmas. Written at the suggestion of @chrisflav , with the following example usecase: ```lean-4 import Mathlib open AlgebraicGeometry attribute [algebraize flat_of_flat] Flat -- pretend this is added where `AlgebraicGeometry.Flat` is defined lemma flat_of_flat {R S : Type u} [CommRing R] [CommRing S] (f : R →+* S) (h : Flat (Spec.map (CommRingCat.ofHom f))) : @Module.Flat R S _ _ f.toAlgebra.toModule := by have : f.Flat := sorry -- supposedly, this is true. ask christian. algebraize [f] assumption set_option tactic.hygienic false -- allow the tactic to produce accessible names for testing example {R S : Type u} [CommRing R] [CommRing S] (f : R →+* S) (h : Flat (Spec.map (CommRingCat.ofHom f))) : True := by algebraize [f] guard_hyp algebraizeInst : Module.Flat R S -- used to fail, succeeds now trivial ``` the key changes that makes this possible are the following: - a different way of making lemma/type applications, creating a term which can be added to the context - a different way of checking that the previously mentioned term actually relevant w/r/t the arguments provided to the tactic The previous check was ad-hoc and flimsy, making requirements of the precise order and the types of the arguments of lemmas or definitions, which resulted in the lemma being applicable in limited cases only. Now we still have some requirements, but these are less stringent. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta awaiting-author enhancement 147/62 Mathlib/Tactic/Algebraize.lean,MathlibTest/algebraize.lean 2 34 ['callesonne', 'chrisflav', 'edegeltje', 'github-actions'] nobody
2-35124
2 days ago
2-35124
2 days ago
26-65389
26 days
25094 grunweg
author:grunweg
feat(Tactic/Positivity): extend EReal support for numeric casts Extend `pos_of_isNat` and `nonneg_of_isNat` to cover monoids which are not necessarily semirings, like EReal. [Zulip discussion](https://leanprover.zulipchat.com/#narrow/channel/113488-general/topic/.22Missing.20Tactics.22.20list/near/519660424) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta awaiting-author 70/36 Mathlib/Tactic/Positivity/Core.lean,MathlibTest/positivity.lean 2 19 ['Paul-Lez', 'YaelDillies', 'github-actions', 'grunweg', 'leanprover-bot', 'leanprover-community-bot-assistant', 'leanprover-community-mathlib4-bot'] nobody
2-34924
2 days ago
2-34924
2 days ago
13-6021
13 days
23658 grunweg
author:grunweg
feat: require that real or complex models with corners have convex interior Follow-up to #18403. --- - [x] depends on: #23657 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-zulip t-differential-geometry WIP 116/18 Mathlib/Geometry/Manifold/Instances/Real.lean,Mathlib/Geometry/Manifold/IsManifold/Basic.lean 2 5 ['github-actions', 'grunweg', 'mathlib4-dependent-issues-bot', 'sgouezel'] nobody
2-31025
2 days ago
6-14472
6 days ago
0-9
9 seconds
17781 robin-carlier
author:robin-carlier
feat(CategoryTheory/Limits/Sifted): characterization of sifted categories Characterize small sifted as those for which the `Type`-valued colimit functor preserves finite product. Deduce that filtered categories, and that categories admitting a final functor from a sifted categories are also sifted. --- Second part of what used to be #17554. The core of the proof relies on a few private lemmas/defs (`colimBoxIsoColimTensColim` and `factorization_prod_comparison_colim` being the most important ones) and I don’t know if that can be avoided. I am still unsure wether or not the part relating sifted categories to filtered categories should be split off in a different file to avoid importing `CategoryTheory/Limits/FilteredColimitCommutesFiniteLimit.lean` every time `CategoryTheory/Limits/Sifted.lean` is imported. The fact that filtered categories are sifted can also be proved without the characterization in this PR (it reduces essentially to `IsFiltered.bowtie`), and so it could also stay in this file with less imports, but I find it nicer to do it using the characterization. - [x] depends on: #17766 - [x] depends on: #17779 - [ ] depends on: #24711 - [ ] depends on: #24686 - [ ] depends on: #24703 - [x] depends on: #24735 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) file-removed t-category-theory blocked-by-other-PR 709/26 Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Monoidal/Closed.lean,Mathlib/CategoryTheory/Closed/Functor.lean,Mathlib/CategoryTheory/Closed/Monoidal.lean,Mathlib/CategoryTheory/Limits/Indization/FilteredColimits.lean,Mathlib/CategoryTheory/Limits/Preserves/Bifunctor.lean,Mathlib/CategoryTheory/Limits/Sifted.lean,Mathlib/CategoryTheory/Monoidal/Bimod.lean,Mathlib/CategoryTheory/Monoidal/Braided/Reflection.lean,Mathlib/CategoryTheory/Monoidal/Category.lean,Mathlib/CategoryTheory/Monoidal/ExternalProduct.lean,Mathlib/CategoryTheory/Monoidal/Internal/Limits.lean,Mathlib/CategoryTheory/Monoidal/Limits/Basic.lean,Mathlib/CategoryTheory/Monoidal/Limits/Preserves.lean 14 9 ['github-actions', 'joelriou', 'mathlib4-dependent-issues-bot'] nobody
2-30944
2 days ago
31-21619
1 month ago
33-11296
33 days
25549 yuma-mizuno
author:yuma-mizuno
refactor(CategoryTheory/Monoidal): define `Mon_.Hom` using type class `IsMon_Hom` This PR changes ```lean structure Mon_.Hom (M N : Mon_ C) where hom : M.X ⟶ N.X one_hom : η ≫ hom = η := by aesop_cat mul_hom : μ ≫ hom = (hom ⊗ hom) ≫ μ := by aesop_cat ``` to ```lean structure Mon_.Hom (M N : Mon_ C) where hom : M.X ⟶ N.X [is_mon_hom : IsMon_Hom hom] ``` and similarly for `Comon_.Hom`. The discussion on Zulip: [#mathlib4 > Refactoring Mod_? @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Refactoring.20Mod_.3F/near/522782252) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory 209/173 Mathlib/Algebra/Category/CoalgCat/ComonEquivalence.lean,Mathlib/CategoryTheory/Monad/EquivMon.lean,Mathlib/CategoryTheory/Monoidal/Bimon_.lean,Mathlib/CategoryTheory/Monoidal/Cartesian/Comon_.lean,Mathlib/CategoryTheory/Monoidal/Cartesian/Mon_.lean,Mathlib/CategoryTheory/Monoidal/CommGrp_.lean,Mathlib/CategoryTheory/Monoidal/CommMon_.lean,Mathlib/CategoryTheory/Monoidal/Comon_.lean,Mathlib/CategoryTheory/Monoidal/Grp_.lean,Mathlib/CategoryTheory/Monoidal/Internal/FunctorCategory.lean,Mathlib/CategoryTheory/Monoidal/Internal/Limits.lean,Mathlib/CategoryTheory/Monoidal/Internal/Module.lean,Mathlib/CategoryTheory/Monoidal/Internal/Types/Basic.lean,Mathlib/CategoryTheory/Monoidal/Mod_.lean,Mathlib/CategoryTheory/Monoidal/Mon_.lean,Mathlib/CategoryTheory/Preadditive/CommGrp_.lean 16 4 ['github-actions', 'leanprover-bot', 'mattrobball'] nobody
2-30089
2 days ago
2-79904
2 days ago
2-79948
2 days
18725 joelriou
author:joelriou
feat(LinearAlgebra): generators of pi tensor products --- - [x] depends on: #18534 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) file-removed t-algebra WIP
label:t-algebra$
252/4 Mathlib.lean,Mathlib/Analysis/NormedSpace/PiTensorProduct/ProjectiveSeminorm.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 8 5 ['github-actions', 'joelriou', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
2-26878
2 days ago
22-31165
22 days ago
0-0
0 seconds
24809 robin-carlier
author:robin-carlier
feat(CategoryTheory/Functor/KanExtension): preservations of Kan extensions Introduce a typeclass `G.PreservesLeftKanExtension F L` that asserts that a functor `G` preserves the left Kan extension of `F` along a functor `L`. Introduce a pointwise variant, and relate it to the non-pointwise version when pointwise extensions exist. Show that a functor that preserves the relevant colimits preserve pointwise left Kan extensions. Construct isomorphisms `L.leftKanExtension F ⋙ G ≅ L.leftKanExtension (F ⋙ G)` when `G.PreservesLeftKanExtension F L` holds. Also construct a functorial version, as an isomorphism `L.lan ⋙ (whiskeringRight _ _ _).obj G ≅ (whiskeringRight _ _ _).obj G ⋙ L.lan`. All results are dualised to right Kan extensions. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory 551/0 Mathlib.lean,Mathlib/CategoryTheory/Functor/KanExtension/Basic.lean,Mathlib/CategoryTheory/Functor/KanExtension/Preserves.lean 3 5 ['TwoFX', 'github-actions', 'joelriou', 'robin-carlier'] nobody
2-25051
2 days ago
28-28334
28 days ago
28-28383
28 days
18285 callesonne
author:callesonne
feat(Bicategory/Grothendieck): functoriality of the grothendieck construction This PR is the start towards proving functoriality of the Grothendieck construction. --- - [x] depends on: #18252 - [x] depends on: #18253 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory 150/13 Mathlib/CategoryTheory/Bicategory/Functor/Pseudofunctor.lean,Mathlib/CategoryTheory/Bicategory/Grothendieck.lean,Mathlib/CategoryTheory/Bicategory/NaturalTransformation/Pseudo.lean,Mathlib/CategoryTheory/Category/Cat.lean 4 n/a ['callesonne', 'github-actions', 'joelriou', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
2-21881
2 days ago
unknown
unknown
24578 b-mehta
author:b-mehta
feat(Pointwise): cardinality of product set in GroupWithZero This PR: * generalises the assumptions to `card_le_card_image₂_left` and `card_le_card_image₂_right` and golf these: they previously required injectivity everywhere despite using it in only one place. (These lemmas were also used in exactly one place each in mathlib) * adds `card_le_card_mul_left_of_injective` and `card_le_card_mul_right_of_injective` which generalise the typeclass assumptions on the existing `card_le_card_mul_left` and `card_le_card_mul_right` * uses the above to add versions of `card_le_card_mul_left` and `card_le_card_mul_right` in groups with zero. This is useful for applying the pointwise constructions to fields In fact, the first versions of all the above lemmas were written in this generality, but that was seemingly lost during an upstream. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
54/16 Mathlib/Algebra/Group/Pointwise/Finset/Basic.lean,Mathlib/Algebra/GroupWithZero/Pointwise/Finset.lean,Mathlib/Data/Finset/NAry.lean 3 1 ['github-actions'] mariainesdff
assignee:mariainesdff
2-20790
2 days ago
32-33368
1 month ago
36-70971
36 days
18254 callesonne
author:callesonne
feat(Bicategory/Modification/Pseudo): define modifications between strong natural transformations of pseudofunctors This PR adds modifications between strong natural transformations of pseudofunctors. At the same time, it improves the existing code on modifications between oplax natural tranformations of oplax functors (by removing some simp lemmas). --- - [x] depends on: #18250 - [x] depends on: #18252 - [x] depends on: #18253 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory 295/60 Mathlib.lean,Mathlib/CategoryTheory/Bicategory/Modification/Oplax.lean,Mathlib/CategoryTheory/Bicategory/Modification/Pseudo.lean,Mathlib/CategoryTheory/Bicategory/NaturalTransformation/Oplax.lean,Mathlib/CategoryTheory/Bicategory/NaturalTransformation/Pseudo.lean 5 12 ['callesonne', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'robin-carlier'] nobody
2-17800
2 days ago
2-17807
2 days ago
24-8616
24 days
21965 JovanGerb
author:JovanGerb
feat: extensible `push`(_neg) tactic - part 1 This is the first part of #21769, namely defining the new tactic, and only tagging the lemmas that have to be tagged to match the old behaviour. This includes - The `push_neg` tactic, which is a macro for `push Not` - The `push` tactic - The `↓pushNeg` simproc that can be used as `simp [↓pushNeg]` - The `push` and `push_neg` tactics in `conv` mode. - The `#push_discr_tree` command to help see what lemmas the tactic is using for a given constant. There are two new files: `Mathlib.Tactic.Push` and `Mathlib.Tactic.Push.Attr`. The latter only introduces the `@[push]` attribute, so that it can be used by early Mathlib files without having to import `Mathlib.Tactic.Push`. Zulip conversation: https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/I.20made.20an.20extensible.20.60push.60.20tactic.20generalizing.20.60push_neg.60/near/499492535 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta 312/185 Mathlib.lean,Mathlib/Combinatorics/SimpleGraph/Extremal/Basic.lean,Mathlib/Data/Nat/Basic.lean,Mathlib/Data/Set/Basic.lean,Mathlib/Order/Defs/LinearOrder.lean,Mathlib/RingTheory/AlgebraicIndependent/TranscendenceBasis.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Push.lean,Mathlib/Tactic/Push/Attr.lean,MathlibTest/push_neg.lean,scripts/noshake.json 11 9 ['JovanGerb', 'github-actions', 'grunweg', 'leanprover-bot', 'leanprover-community-bot-assistant'] robertylewis
assignee:robertylewis
2-17362
2 days ago
2-17387
2 days ago
110-71073
110 days
25338 wwylele
author:wwylele
feat(GroupTheory): add divisible completion This is part of #25140. In order to "decompose" a linearly ordered group by its Archimedean classes, it needs to be embedded in a divisible group first. This code prepares for that embedding. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
372/0 Mathlib.lean,Mathlib/GroupTheory/DivisibleCompletion.lean 2 1 ['github-actions'] nobody
2-12682
2 days ago
2-12682
2 days ago
0-0
0 seconds
25543 FrankieNC
author:FrankieNC
feat(MeasureTheory/Measure): bound Hausdorff measure under orthogonal projection Formalisation that Hausdorff measure is non-increasing under orthogonal projection onto a finite-dimensional Euclidean subspace. This includes: * a bound on the norm of orthogonal projections; * a proof that orthogonal projection is 1-Lipschitz; * the main result: the `s`-dimensional Hausdorff measure of the projection of a set is less than or equal to that of the original set. This formalises Lemma 3.5 from Julian Fox’s REU paper: *Besicovitch Sets, Kakeya Sets, and Their Properties*, UChicago REU, 2021. --- Footer _No breaking changes._ --- Dependencies _None._ --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-measure-probability 43/2 Mathlib/Analysis/InnerProductSpace/Projection.lean,Mathlib/MeasureTheory/Measure/Hausdorff.lean 2 9 ['b-mehta', 'github-actions'] nobody
2-11991
2 days ago
2-79905
2 days ago
3-6633
3 days
25331 fbarroero
author:fbarroero
feat(RingTheory/Ideal/Maximal): `ne_top_iff_exists_maximal` We add `Ideal.ne_top_iff_exists_maximal` and an analogous statement for `IsDedekindDomain.HeightOneSpectrum`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
18/0 Mathlib/RingTheory/DedekindDomain/Ideal.lean,Mathlib/RingTheory/Ideal/Maximal.lean 2 5 ['Ruben-VandeVelde', 'fbarroero', 'github-actions'] nobody
2-7027
2 days ago
9-18489
9 days ago
9-18541
9 days
14089 callesonne
author:callesonne
feat(Bicategory/Functorbicategory): define bicategory of pseudofunctors This PR contains a definition of the bicategory of pseudofunctors, in the file `Bicategory/FunctorBicategory/Pseudo.lean`. It also moves the file `Bicategory/Functorbicategory.lean` to `Bicategory/FunctorBicategory/Oplax.lean`. --- - [x] depends on: #14028 - [x] depends on: #18250 - [x] depends on: #18252 - [x] depends on: #18253 - [ ] depends on: #18254 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory blocked-by-other-PR 385/70 Mathlib.lean,Mathlib/CategoryTheory/Bicategory/FunctorBicategory/Oplax.lean,Mathlib/CategoryTheory/Bicategory/FunctorBicategory/Pseudo.lean,Mathlib/CategoryTheory/Bicategory/Modification/Oplax.lean,Mathlib/CategoryTheory/Bicategory/Modification/Pseudo.lean,Mathlib/CategoryTheory/Bicategory/NaturalTransformation/Oplax.lean,Mathlib/CategoryTheory/Bicategory/NaturalTransformation/Pseudo.lean 7 5 ['callesonne', 'github-actions', 'leanprover-community-bot-assistant', 'leanprover-community-mathlib4-bot'] nobody
2-4615
2 days ago
2-5993
2 days ago
9-2320
9 days
23929 meithecatte
author:meithecatte
feat(Computability/NFA): improve bound on pumping lemma --- - [x] depends on: #25321 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-zulip t-computability new-contributor 101/10 Mathlib/Computability/EpsilonNFA.lean,Mathlib/Computability/NFA.lean 2 41 ['YaelDillies', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'meithecatte'] nobody
2-1067
2 days ago
2-1068
2 days ago
34-10595
34 days
25089 Bergschaf
author:Bergschaf
feat(Order/Sublocale): definition of sublocales There are several possible definition of sublocales. I used one from [nlab](https://ncatlab.org/nlab/show/sublocale) which states that a sublocale is a subset of a locale which is closed under all meets and for any ∈ S and x ∈ X, we have x ⇨ s ∈ S. This PR also includes an order isomorphism between (Nucleus)ᵒᵈ and Sublocale. --- I am open to better name suggestions for the order isomorphism. - [x] depends on: #24941 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) maintainer-merge t-order 265/8 Mathlib.lean,Mathlib/Order/Hom/Lattice.lean,Mathlib/Order/Nucleus.lean,Mathlib/Order/Sublocale.lean,Mathlib/Order/Synonym.lean,docs/references.bib 6 71 ['Bergschaf', 'YaelDillies', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'xhalo32'] nobody
2-955
2 days ago
2-955
2 days ago
15-66778
15 days
25501 eric-wieser
author:eric-wieser
fix: eliminate metadata in linarith Otherwise this interferes with the `answer()` elaborator from formal-conjectures. Diagnosed using #25500. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta delegated bug 7/1 Mathlib/Tactic/Linarith/Parsing.lean,MathlibTest/linarith.lean 2 8 ['adomani', 'b-mehta', 'github-actions', 'j-loreaux', 'leanprover-bot', 'mathlib-bors'] nobody
1-85708
1 day ago
2-1462
2 days ago
1-78612
1 day
25350 thorimur
author:thorimur
feat: add autoparams for proof fields of `Equiv` This PR adds the simple autoparam `by intro; first | rfl | ext <;> rfl` for the fields `left_inv`, `right_inv` of `Equiv`, and removes explicit terms in favor of the autoparam across mathlib in many (but possibly not all) applicable cases. It also adds the same autoparam to the corresponding fields of `LieEquiv` for parity (which is used nontrivially in `LieSubalgebra.topEquiv` in `Mathlib.Algebra.Lie.Submodule`). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-logic 39/653 Counterexamples/AharoniKorman.lean,Mathlib/Algebra/AddConstMap/Equiv.lean,Mathlib/Algebra/Algebra/Basic.lean,Mathlib/Algebra/Algebra/Equiv.lean,Mathlib/Algebra/Algebra/NonUnitalHom.lean,Mathlib/Algebra/Algebra/Opposite.lean,Mathlib/Algebra/Algebra/Prod.lean,Mathlib/Algebra/Algebra/Spectrum/Pi.lean,Mathlib/Algebra/Algebra/Spectrum/Quasispectrum.lean,Mathlib/Algebra/Category/CommAlgCat/Basic.lean,Mathlib/Algebra/Category/Grp/Adjunctions.lean,Mathlib/Algebra/Category/ModuleCat/Basic.lean,Mathlib/Algebra/Category/ModuleCat/ChangeOfRings.lean,Mathlib/Algebra/Category/ModuleCat/Monoidal/Closed.lean,Mathlib/Algebra/Category/ModuleCat/Sheaf/ChangeOfRings.lean,Mathlib/Algebra/DualQuaternion.lean,Mathlib/Algebra/Free.lean,Mathlib/Algebra/FreeMonoid/Basic.lean,Mathlib/Algebra/Group/AddChar.lean,Mathlib/Algebra/Group/End.lean,Mathlib/Algebra/Group/Equiv/Opposite.lean,Mathlib/Algebra/Group/Equiv/TypeTags.lean,Mathlib/Algebra/Group/Pi/Units.lean,Mathlib/Algebra/Group/Subgroup/Map.lean,Mathlib/Algebra/Group/Submonoid/Operations.lean,Mathlib/Algebra/Group/Submonoid/Units.lean,Mathlib/Algebra/Group/Subsemigroup/Operations.lean,Mathlib/Algebra/Group/TypeTags/Hom.lean,Mathlib/Algebra/Group/Units/Equiv.lean,Mathlib/Algebra/Group/Units/Opposite.lean,Mathlib/Algebra/Group/WithOne/Basic.lean,Mathlib/Algebra/GroupWithZero/Action/Center.lean,Mathlib/Algebra/GroupWithZero/NonZeroDivisors.lean,Mathlib/Algebra/GroupWithZero/Units/Equiv.lean,Mathlib/Algebra/GroupWithZero/WithZero.lean,Mathlib/Algebra/Homology/ComplexShapeSigns.lean,Mathlib/Algebra/Homology/Square.lean,Mathlib/Algebra/Lie/Basic.lean,Mathlib/Algebra/Lie/Character.lean,Mathlib/Algebra/Lie/Submodule.lean,Mathlib/Algebra/Module/Equiv/Basic.lean,Mathlib/Algebra/Module/Presentation/DirectSum.lean,Mathlib/Algebra/Module/Presentation/Tautological.lean,Mathlib/Algebra/Module/Submodule/Equiv.lean,Mathlib/Algebra/Module/Submodule/Lattice.lean,Mathlib/Algebra/Module/Submodule/Map.lean,Mathlib/Algebra/Module/ZMod.lean,Mathlib/Algebra/Order/Antidiag/Prod.lean,Mathlib/Algebra/Order/Ring/Idempotent.lean,Mathlib/Algebra/Polynomial/Basic.lean,Mathlib/Algebra/Polynomial/Module/AEval.lean,Mathlib/Algebra/Quandle.lean,Mathlib/Algebra/Quaternion.lean,Mathlib/Algebra/Ring/Equiv.lean,Mathlib/Algebra/Ring/Opposite.lean,Mathlib/Algebra/Ring/Prod.lean,Mathlib/Algebra/Ring/Subsemiring/Basic.lean,Mathlib/Algebra/SkewMonoidAlgebra/Basic.lean,Mathlib/Algebra/Star/StarAlgHom.lean,Mathlib/Algebra/TrivSqZeroExt.lean,Mathlib/AlgebraicGeometry/PointsPi.lean,Mathlib/AlgebraicTopology/FundamentalGroupoid/Basic.lean,Mathlib/AlgebraicTopology/SimplicialSet/HomotopyCat.lean,Mathlib/AlgebraicTopology/SimplicialSet/Nerve.lean,Mathlib/AlgebraicTopology/SimplicialSet/StdSimplex.lean,Mathlib/Analysis/BoxIntegral/Partition/Filter.lean,Mathlib/Analysis/InnerProductSpace/Adjoint.lean,Mathlib/Analysis/Normed/Algebra/Spectrum.lean,Mathlib/Analysis/Normed/Group/Hom.lean,Mathlib/Analysis/Normed/Group/SeparationQuotient.lean,Mathlib/Analysis/Normed/Lp/LpEquiv.lean,Mathlib/Analysis/NormedSpace/Alternating/Basic.lean,Mathlib/Analysis/NormedSpace/Multilinear/Curry.lean,Mathlib/CategoryTheory/Category/Bipointed.lean,Mathlib/CategoryTheory/Category/Cat/Adjunction.lean,Mathlib/CategoryTheory/Category/Pointed.lean,Mathlib/CategoryTheory/Category/TwoP.lean,Mathlib/CategoryTheory/CodiscreteCategory.lean,Mathlib/CategoryTheory/CofilteredSystem.lean,Mathlib/CategoryTheory/Comma/Arrow.lean,Mathlib/CategoryTheory/Comma/CardinalArrow.lean,Mathlib/CategoryTheory/Endomorphism.lean,Mathlib/CategoryTheory/Enriched/Basic.lean,Mathlib/CategoryTheory/Functor/FunctorHom.lean,Mathlib/CategoryTheory/Functor/TwoSquare.lean,Mathlib/CategoryTheory/GradedObject/Trifunctor.lean,Mathlib/CategoryTheory/Groupoid.lean,Mathlib/CategoryTheory/Limits/Preserves/Ulift.lean,Mathlib/CategoryTheory/Limits/Shapes/SingleObj.lean,Mathlib/CategoryTheory/Limits/Types/Shapes.lean,Mathlib/CategoryTheory/Limits/Types/Yoneda.lean,Mathlib/CategoryTheory/Localization/Construction.lean,Mathlib/CategoryTheory/Localization/Resolution.lean,Mathlib/CategoryTheory/Monad/Monadicity.lean,Mathlib/CategoryTheory/Opposites.lean,Mathlib/CategoryTheory/Sites/Sheaf.lean,Mathlib/CategoryTheory/Sites/SheafHom.lean,Mathlib/CategoryTheory/Yoneda.lean,Mathlib/Combinatorics/Configuration.lean,Mathlib/Combinatorics/Quiver/Basic.lean 219 11 ['JovanGerb', 'adomani', 'github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'leanprover-community-mathlib4-bot', 'thorimur'] nobody
1-85034
1 day ago
2-1832
2 days ago
3-58230
3 days
25480 ocfnash
author:ocfnash
feat: define a concrete model of the `𝔤₂` root system This is a bit of an experiment to test API but it should also make it easier to prove some properties of `𝔤₂`. --- - [x] depends on: #25477 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-algebra WIP
label:t-algebra$
50/0 Mathlib/LinearAlgebra/RootSystem/Finite/G2.lean 1 7 ['eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'ocfnash'] nobody
1-84505
1 day ago
1-84523
1 day ago
0-1
1 second
25565 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/) t-category-theory 286/0 Mathlib.lean,Mathlib/CategoryTheory/Bicategory/NaturalTransformation/Lax.lean,scripts/noshake.json 3 13 ['callesonne', 'github-actions', 'robin-carlier', 'yuma-mizuno'] nobody
1-72993
1 day ago
1-77544
1 day ago
2-12525
2 days
25575 Rida-Hamadani
author:Rida-Hamadani
feat(SimpleGraph): ext for walks based on `getVert` and `support` Two walks are the same if they agree under `getVert` or `support`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics 43/0 Mathlib/Combinatorics/SimpleGraph/Walk.lean 1 6 ['Rida-Hamadani', 'b-mehta', 'github-actions'] nobody
1-64605
1 day ago
1-65815
1 day ago
1-69165
1 day
25495 adomani
author:adomani
chore: use non-deprecated function in bench_summary Discovered while investigating why the bot has been failing recently: this will likely not fix the bot, but should be updated anyway! --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 1/1 scripts/bench_summary.lean 1 4 ['github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot'] nobody
1-50302
1 day ago
4-9243
4 days ago
4-12357
4 days
25481 kbuzzard
author:kbuzzard
chore: refactor Algebra.TensorProduct.rightAlgebra The declaration `Algebra.TensorProduct.rightAlgebra` makes `A ⊗[R] B` into a `B`-algebra (here `R` is a `CommSemiring`, `A` is a `Semiring` and an `R`-algebra, and `B` is a `CommSemiring` and an `R`-algebra). It is not an instance because if A = B it causes a diamond. However in the many cases where A isn't B, it can occasionally be useful. However one could imagine that in the many cases where an R-module `M` also isn't `B`, it might occasionally be useful to make `M ⊗[R] B` into a `B`-module (and indeed I am finding this in FLT). With the current definition of `Algebra.TensorProduct.rightAlgebra` this is difficult to do without causing diamonds in the case when `M` happens to be an `R`-algebra (by which I mean "I failed to do this in finite time"). One fix for this is just to redefine `Algebra.TensorProduct.rightAlgebra` so that the `smul` field is ``` smul b ab := TensorProduct.comm _ _ _ (b • (TensorProduct.comm _ _ _ ab)) ``` i.e. literally "swap the product around, use mathlib's instance making `B ⊗[R] A` into a `B`-algebra, and then swap back". Then the same definition can be used to make `M ⊗[R] B` into a `B`-module and on the odd occasion where this point of view is useful, there is no diamond. This is what we do in this PR. After adding one simp lemma there is no breakage at all in mathlib. Furthermore, for those who have observed that we want to build on this algebra instance sometimes and, for example, add instances of the form "if M is finite over R then M ⊗[R] B is finite over B" -- these instances are really easy to add now with this new definition, because you simply pull back the analogous finite left module instance along the isomorphism M ⊗[R] B = B ⊗[R] M. Examples (from FLT, where the right action is put in a scope): ``` scoped instance [Module.Finite R M] : Module.Finite A (M ⊗[R] A) := Module.Finite.equiv (Module.TensorProduct.comm R A M) scoped instance [Module.Free R M] : Module.Free A (M ⊗[R] A) := Module.Free.of_equiv (Module.TensorProduct.comm R A M) ``` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
33/6 Mathlib/RingTheory/TensorProduct/Basic.lean 1 4 ['github-actions', 'kbuzzard', 'leanprover-bot'] nobody
1-43742
1 day ago
4-23289
4 days ago
4-23547
4 days
24149 YaelDillies
author:YaelDillies
refactor(Convex/Cone): reorder, streamline The current library on cones is very centered around normed and Hilbert spaces. This is inconvenient for us in Toric where we have two spaces $M$, and $N$ that are non-canonically isomorphic to $ℐ R^n$ (for the same $n$). Although we could identify $M$ and $N$ with $ℐ R^n$ and get an inner product on $M = N = ℐ R^n$ this way, we would lose the contravariance (resp. covariance) of $M$ (resp. $N$) in the group scheme that indexes them. We would instead like to have results that apply to perfect pairings $p : M → N → ℐ R$ out of the box. Not all the theory can be generalised, of course. So, in terms of file structure, we need to draw the line somewhere. We propose to draw it at the import of `NormedAddCommGroup`, as this is the time where the scalars suddenly get fixed to the reals, instead of an arbitrary ordered ring. This line passes through individual files, which therefore need to be split. We operate this separation by moving the cone content that doesn't require a norm under a new folder `Geometry.Convex.Cone`. The content that does require it stays in `Analysis.Convex.Cone`. A similar operation could be performed for the rest of the `Analysis.Convex`, but it seems wiser to do so simultaneously with the convexity refactor. Changes performed include: * Renaming the variable `𝕜` to `R` when it is merely a ring * Splitting files according to normless normful parts * Completing the existing APIs * Redefining `ProperCone R M` as an `abbrev` for `ClosedSubmodule R≥0 M`, similarly to how `PointedCone R M` is an `abbrev` for `Submodule R≥0 M`. * Replacing the three dual cones definitions we have: * `Set.innerDualCone : Set H → ConvexCone ℝ H` * `PointedCone.dual : PointedCone ℝ H → PointedCone ℝ H` * `ProperCone.dual : ProperCone ℝ H → ProperCone ℝ H` by three new ones: * `PointedCone.dual : Set M → PointedCone R N` for a bilinear pairing `p : M →ₗ[R] N →ₗ[R] R` * `ProperCone.dual : Set M → ProperCone R N` for a continuous perfect pairing `p : M →ₗ[R] N →ₗ[R] R` * `ProperCone.innerDual : Set H → ProperCone ℝ H` for an inner product space `H` From Toric --- - [x] depends on: #24229 - [x] depends on: #24230 - [x] depends on: #24231 - [x] depends on: #24232 - [x] depends on: #24233 - [x] depends on: #24234 - [x] depends on: #24235 - [x] depends on: #24236 - [x] depends on: #24237 - [ ] depends on: #24304 - [ ] depends on: #25204 - [ ] depends on: #25251 - [x] depends on: #25252 - [ ] depends on: #25292 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) file-removed toric large-import new-contributor t-analysis blocked-by-other-PR 1072/909 Mathlib.lean,Mathlib/Analysis/Convex/Cone/Basic.lean,Mathlib/Analysis/Convex/Cone/Closure.lean,Mathlib/Analysis/Convex/Cone/Dual.lean,Mathlib/Analysis/Convex/Cone/Extension.lean,Mathlib/Analysis/Convex/Cone/InnerDual.lean,Mathlib/Analysis/Convex/Cone/Pointed.lean,Mathlib/Analysis/Convex/Cone/Proper.lean,Mathlib/Analysis/Convex/Cone/README.md,Mathlib/Geometry/Convex/Cone/Basic.lean,Mathlib/Geometry/Convex/Cone/Dual.lean,Mathlib/Geometry/Convex/Cone/Pointed.lean,Mathlib/Geometry/Convex/Cone/README.md,Mathlib/Topology/Algebra/Module/PerfectPairing.lean 14 13 ['YaelDillies', 'github-actions', 'justus-springer', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
1-43736
1 day ago
1-43754
1 day ago
1-83310
1 day
25558 kbuzzard
author:kbuzzard
chore: split Mathlib/Topology/Algebra/RestrictedProduct `Mathlib/Topology/Algebra/RestrictedProduct.lean` is over 1000 lines and we have over 500 lines more of restricted product API in FLT with more to come, so I thought I would split sooner rather than later. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) This PR is nothing more than a split with no additions or deletions. file-removed t-topology 408/360 Mathlib.lean,Mathlib/RingTheory/DedekindDomain/FiniteAdeleRing.lean,Mathlib/Topology/Algebra/RestrictedProduct/Basic.lean,Mathlib/Topology/Algebra/RestrictedProduct/TopologicalSpace.lean,scripts/noshake.json 5 4 ['eric-wieser', 'github-actions', 'grunweg', 'kbuzzard'] nobody
1-43081
1 day ago
2-39635
2 days ago
2-39689
2 days
25563 Komyyy
author:Komyyy
chore: move `Topology.StoneCech` into `Topology.Compactification` (1/2) At present, the `Topology.Compactification` directory includes results on one-point compactifications, but results on Stone-Čech compactifications are currently located elsewhere. The removed file `Topology.Compactification` is deprecated in another PR (#25583) to leave a good git diff history. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) file-removed maintainer-merge t-topology 9/9 Mathlib.lean,Mathlib/Combinatorics/Hindman.lean,Mathlib/Topology/Category/CompHaus/Basic.lean,Mathlib/Topology/Category/CompHaus/Projective.lean,Mathlib/Topology/Category/Profinite/Projective.lean,Mathlib/Topology/Category/Stonean/Adjunctions.lean,Mathlib/Topology/Compactification/StoneCech.lean,Mathlib/Topology/ExtremallyDisconnected.lean,Mathlib/Topology/Maps/Proper/UniversallyClosed.lean,Mathlib/Topology/Separation/CompletelyRegular.lean 10 4 ['Komyyy', 'github-actions', 'grunweg'] nobody
1-42111
1 day ago
1-42111
1 day ago
2-17644
2 days
25561 callesonne
author:callesonne
feat(Category/Grpd): define the bicategory of groupoids --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory 179/25 Mathlib.lean,Mathlib/AlgebraicTopology/FundamentalGroupoid/InducedMaps.lean,Mathlib/CategoryTheory/Bicategory/Functor/Pseudofunctor.lean,Mathlib/CategoryTheory/Bicategory/Functor/Strict.lean,Mathlib/CategoryTheory/Category/Cat.lean,Mathlib/CategoryTheory/Category/Grpd.lean 6 4 ['callesonne', 'github-actions', 'robin-carlier'] nobody
1-41265
1 day ago
1-85841
1 day ago
2-19997
2 days
24330 Paul-Lez
author:Paul-Lez
chore(Data/Nat/Factorization/Basic): minimize dependencies --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data WIP 123/103 Mathlib.lean,Mathlib/Algebra/Order/Antidiag/Nat.lean,Mathlib/Data/Nat/Factorization/Basic.lean,Mathlib/Data/Nat/Factorization/Defs.lean,Mathlib/Data/Nat/Factorization/LCM.lean,Mathlib/Data/Nat/Multiplicity.lean,Mathlib/GroupTheory/Exponent.lean,Mathlib/NumberTheory/Cyclotomic/PrimitiveRoots.lean,Mathlib/RingTheory/RootsOfUnity/PrimitiveRoots.lean 9 5 ['YaelDillies', 'github-actions', 'leanprover-community-bot-assistant'] YaelDillies
assignee:YaelDillies
1-40316
1 day ago
1-43556
1 day ago
0-0
0 seconds
21871 YaelDillies
author:YaelDillies
feat: decomposition into independent atoms Prove that any element in a compactly generated modular atomistic lattice (eg the lattice of submodules of a module) can be written as the supremum of independent atoms. From PersistentDecomp and Xena --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order help-wanted 113/20 Mathlib/Data/Set/Insert.lean,Mathlib/Order/Atoms.lean,Mathlib/Order/CompactlyGenerated/Basic.lean 3 3 ['github-actions', 'leanprover-community-bot-assistant'] nobody
1-39562
1 day ago
1-39585
1 day ago
0-15
15 seconds
24384 joelriou
author:joelriou
feat(CategoryTheory): pseudofunctors to Cat We specialize the API from PR #24382 to the case of pseudofunctors to `Cat`. Co-authored-by: Christian Merten [christian@merten.dev](mailto:christian@merten.dev) --- - [ ] depends on: #24382 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory awaiting-author blocked-by-other-PR 359/0 Mathlib.lean,Mathlib/CategoryTheory/Bicategory/Functor/Cat.lean,Mathlib/CategoryTheory/Bicategory/Functor/Strict.lean 3 5 ['callesonne', 'github-actions', 'mathlib4-dependent-issues-bot'] nobody
1-36291
1 day ago
1-75906
1 day ago
0-29
29 seconds
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$
251/185 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/RingTheory/Ideal/Quotient/Index.lean 14 22 ['Ruben-VandeVelde', 'TwoFX', 'YaelDillies', 'alreadydone', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'loefflerd', 'madvorak', 'mathlib4-dependent-issues-bot', 'tb65536'] nobody
1-34509
1 day ago
1-34662
1 day ago
129-18967
129 days
24913 YaelDillies
author:YaelDillies
feat: if `p = a * b` is irreducible, then `a = 1` or `b = 1` From Toric --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) toric t-algebra
label:t-algebra$
7/3 Mathlib/Algebra/Group/Irreducible/Defs.lean 1 6 ['Ruben-VandeVelde', 'YaelDillies', 'b-mehta', 'github-actions'] nobody
1-34407
1 day ago
1-34467
1 day ago
25-40714
25 days
25579 JovanGerb
author:JovanGerb
feat(Order/Notation): only allow ⊔/⊓ for non-linear orders ⊔/⊓ is the same as max/min. The difference is that it is meant to be used if and only if there is no linear order. This PR implements a check for one of the two directions. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order 33/7 Mathlib/Order/Notation.lean 1 1 ['github-actions'] nobody
1-34175
1 day ago
1-63111
1 day ago
0-0
0 seconds
25580 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 134/125 Mathlib/AlgebraicTopology/DoldKan/Decomposition.lean,Mathlib/AlgebraicTopology/DoldKan/Degeneracies.lean,Mathlib/AlgebraicTopology/DoldKan/NCompGamma.lean,Mathlib/AlgebraicTopology/DoldKan/Projections.lean,Mathlib/AlgebraicTopology/SimplexCategory/MorphismProperty.lean,Mathlib/AlgebraicTopology/SimplicialObject/Split.lean,Mathlib/AlgebraicTopology/SimplicialSet/Degenerate.lean,Mathlib/AlgebraicTopology/SimplicialSet/NerveAdjunction.lean,Mathlib/AlgebraicTopology/SimplicialSet/StdSimplex.lean,Mathlib/CategoryTheory/Abelian/GrothendieckCategory/EnoughInjectives.lean,Mathlib/CategoryTheory/Abelian/GrothendieckCategory/Subobject.lean,Mathlib/CategoryTheory/Action/Concrete.lean,Mathlib/CategoryTheory/Action/Monoidal.lean,Mathlib/CategoryTheory/ComposableArrows.lean,Mathlib/CategoryTheory/Extensive.lean,Mathlib/CategoryTheory/Filtered/Basic.lean,Mathlib/CategoryTheory/Galois/Decomposition.lean,Mathlib/CategoryTheory/Galois/EssSurj.lean,Mathlib/CategoryTheory/Limits/Shapes/Equalizers.lean,Mathlib/CategoryTheory/Limits/Shapes/SequentialProduct.lean,Mathlib/CategoryTheory/Limits/Types/Colimits.lean,Mathlib/CategoryTheory/Limits/VanKampen.lean,Mathlib/CategoryTheory/Quotient.lean,Mathlib/CategoryTheory/Sites/Sheaf.lean,Mathlib/CategoryTheory/Subobject/Basic.lean,Mathlib/CategoryTheory/Subobject/FactorThru.lean,Mathlib/CategoryTheory/Subobject/Lattice.lean,Mathlib/CategoryTheory/Triangulated/TStructure/Basic.lean 28 3 ['Parcly-Taxel', 'eric-wieser', 'github-actions'] nobody
1-30932
1 day ago
1-57008
1 day ago
1-56994
1 day
25174 zcyemi
author:zcyemi
feat(Geometry/Euclidean/Triangle): add law of sines --- Implement the vector and angle-at-point forms of the law of sines. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-euclidean-geometry 57/1 Mathlib/Geometry/Euclidean/Triangle.lean 1 15 ['eric-wieser', 'github-actions', 'jsm28', 'zcyemi'] nobody
1-29741
1 day ago
15-50897
15 days ago
15-50951
15 days
25578 peakpoint
author:peakpoint
refactor(Geometry/Euclidean/Projection): redefine projection and reflection for affine subspaces --- The coersion stuff is just copied from `Analysis/Normed/Operator/LinearIsometry`. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-euclidean-geometry 479/448 Mathlib.lean,Mathlib/Analysis/Normed/Affine/ContinuousAffineMap.lean,Mathlib/Analysis/Normed/Affine/Isometry.lean,Mathlib/Geometry/Euclidean/Altitude.lean,Mathlib/Geometry/Euclidean/Circumcenter.lean,Mathlib/Geometry/Euclidean/Projection.lean,Mathlib/Geometry/Euclidean/SignedDist.lean,Mathlib/LinearAlgebra/AffineSpace/AffineSubspace/Projection.lean 8 2 ['github-actions', 'jsm28'] nobody
1-29273
1 day ago
1-64573
1 day ago
1-64569
1 day
23181 YaelDillies
author:YaelDillies
chore(UniformSpace/Defs): move entourages to their own file 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). --- - [ ] depends on: #25587 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology awaiting-CI blocked-by-other-PR 552/667 Mathlib.lean,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/Topology/Metrizable/Uniformity.lean,Mathlib/Topology/UniformSpace/Defs.lean,Mathlib/Topology/UniformSpace/Entourage.lean 14 20 ['ADedecker', 'PatrickMassot', 'YaelDillies', 'b-mehta', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
1-27151
1 day ago
1-27700
1 day ago
43-40011
43 days
23124 YaelDillies
author:YaelDillies
feat(MetricSpace): nets Define nets, which are a quantitative notion of compactness in a metric space. From my PhD (MiscYD) --- - [x] depends on: #23180 - [ ] depends on: #23181 - [ ] depends on: #23920 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology awaiting-CI blocked-by-other-PR 943/788 Mathlib.lean,Mathlib/CategoryTheory/Category/RelCat.lean,Mathlib/Combinatorics/Hall/Basic.lean,Mathlib/Combinatorics/SimpleGraph/Basic.lean,Mathlib/Combinatorics/SimpleGraph/Path.lean,Mathlib/Combinatorics/SimpleGraph/Subgraph.lean,Mathlib/Data/PFun.lean,Mathlib/Data/Rel.lean,Mathlib/Dynamics/TopologicalEntropy/CoverEntropy.lean,Mathlib/Dynamics/TopologicalEntropy/DynamicalEntourage.lean,Mathlib/Dynamics/TopologicalEntropy/NetEntropy.lean,Mathlib/Dynamics/TopologicalEntropy/Semiconj.lean,Mathlib/Order/Filter/Partial.lean,Mathlib/Order/JordanHolder.lean,Mathlib/Order/KrullDimension.lean,Mathlib/Order/Rel/GaloisConnection.lean,Mathlib/Order/RelSeries.lean,Mathlib/RingTheory/Ideal/AssociatedPrime/Finiteness.lean,Mathlib/RingTheory/Length.lean,Mathlib/RingTheory/Spectrum/Prime/LTSeries.lean,Mathlib/Topology/MetricSpace/Cover.lean,Mathlib/Topology/MetricSpace/MetricSeparated.lean,Mathlib/Topology/Metrizable/Uniformity.lean,Mathlib/Topology/UniformSpace/Basic.lean,Mathlib/Topology/UniformSpace/Cauchy.lean,Mathlib/Topology/UniformSpace/Cover.lean,Mathlib/Topology/UniformSpace/Defs.lean,Mathlib/Topology/UniformSpace/Entourage.lean,Mathlib/Topology/UniformSpace/Separated.lean,Mathlib/Topology/UniformSpace/UniformConvergence.lean 30 15 ['D-Thomine', 'YaelDillies', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'urkud'] nobody
1-27004
1 day ago
1-27020
1 day ago
1-52822
1 day
25583 Komyyy
author:Komyyy
style: move `Topology.StoneCech` into `Topology.Compactification` (2/2) This file deprecates the removed file `Topology.Compactification`. This PR is split from #25563 to leave a good git diff history. --- For reviewers: It's welcome to merge master after #25563 is merged. - [ ] depends on: #25563 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology blocked-by-other-PR 405/393 Mathlib.lean,Mathlib/Combinatorics/Hindman.lean,Mathlib/Topology/Category/CompHaus/Basic.lean,Mathlib/Topology/Category/CompHaus/Projective.lean,Mathlib/Topology/Category/Profinite/Projective.lean,Mathlib/Topology/Category/Stonean/Adjunctions.lean,Mathlib/Topology/Compactification/StoneCech.lean,Mathlib/Topology/ExtremallyDisconnected.lean,Mathlib/Topology/Maps/Proper/UniversallyClosed.lean,Mathlib/Topology/Separation/CompletelyRegular.lean,Mathlib/Topology/StoneCech.lean 11 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
1-22243
1 day ago
1-42718
1 day ago
0-1
1 second
23502 Timeroot
author:Timeroot
feat(ModelTheory/Semantics): BoundedFormula.realize_foldr_imp Two lemmas for `realize`ing a `BoundedFormula`. --- Pulled out from #19695. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-logic 20/0 Mathlib/ModelTheory/Semantics.lean,Mathlib/ModelTheory/Syntax.lean 2 2 ['Timeroot', 'github-actions'] fpvandoorn
assignee:fpvandoorn
1-19362
1 day ago
70-16572
2 months ago
70-16623
70 days
23858 xroblot
author:xroblot
feat(NumberField/CMField): All CM-extensions come from the real maximal subfield Main result: if `K/F` is a CM-extension then `F` is isomorphic to the maximal real subfield of `K` --- - [x] depends on: #23760 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-number-theory 113/6 Mathlib/Algebra/Field/Subfield/Basic.lean,Mathlib/FieldTheory/IntermediateField/Adjoin/Basic.lean,Mathlib/FieldTheory/IntermediateField/Basic.lean,Mathlib/LinearAlgebra/Dimension/Finrank.lean,Mathlib/NumberTheory/NumberField/CMField.lean 5 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
1-17525
1 day ago
2-32914
2 days ago
2-33897
2 days
20924 tomaz1502
author:tomaz1502
feat(Computability/QueryComplexity): Oracle-based computation This PR adds the types and lemmas for oracle-based computation. In this model, computations are run on a monad which also counts the number of oracle queries executed. With it, it becomes possible to reason about the upper bound of the query complexity of algorithms. In the future, we could extend this work to include the necessary bits from information theory and probability to also reason about lower bounds on query complexity, like the work in https://github.com/girving/debate. Zulip discussion: https://leanprover.zulipchat.com/#narrow/channel/144837-PR-reviews/topic/.2318629.20runtime.20complexity.20of.20sorting.20a.20list Co-authored-by: Geoffrey Irving --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-computability 305/0 Mathlib.lean,Mathlib/Computability/QueryComplexity/Basic.lean,Mathlib/Computability/QueryComplexity/Defs.lean 3 58 ['eric-wieser', 'girving', 'github-actions', 'quangvdao', 'tomaz1502'] nobody
1-15090
1 day ago
138-13504
4 months ago
138-13495
138 days
24144 joelriou
author:joelriou
feat(CategoryTheory): the derived adjunction between absolute derived functors An adjunction between functors induces an adjunction between the corresponding left/right derived functors, when these derived functors are *absolute*, i.e. they remain derived functors after the post-composition with any functor. This theorem is the generalized version by Georges Maltsiniotis (*Le théorème de Quillen, d'adjonction des foncteurs dérivés, revisité*, C. R. Math. Acad. Sci. Paris 344 (2007), no. 9) of a theorem by Quillen for adjunctions between model categories. --- - [x] depends on: #24142 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory 159/0 Mathlib.lean,Mathlib/CategoryTheory/Functor/Derived/Adjunction.lean,docs/references.bib 3 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] adamtopaz
assignee:adamtopaz
1-14703
1 day ago
22-81104
22 days ago
22-81087
22 days
25595 joelriou
author:joelriou
feat(CategoryTheory/Bicategory): more compatibilities for mates This PR shows some additional compatibilities for mates in bicategories. It shall be used in the construction of the bicategory of adjunctions in a bicategory #13539. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory 103/0 Mathlib/CategoryTheory/Bicategory/Adjunction/Mate.lean 1 1 ['github-actions'] nobody
1-13757
1 day ago
1-13831
1 day ago
1-13817
1 day
13539 joelriou
author:joelriou
feat: the bicategory of adjunctions in a bicategory --- - [x] depends on: #24982 - [ ] depends on: #25595 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory blocked-by-other-PR 336/0 Mathlib.lean,Mathlib/CategoryTheory/Bicategory/Adjunction/Adj.lean,Mathlib/CategoryTheory/Bicategory/Adjunction/Mate.lean 3 4 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'riccardobrasca'] nobody
1-13273
1 day ago
1-13274
1 day ago
1-18200
1 day
24382 joelriou
author:joelriou
feat(CategoryTheory): pseudofunctors from strict bicategories This PR provides an API for pseudofunctors `F` from a strict bicategory `B`. In particular, this shall apply to pseudofunctors from locally discrete bicategories. We first introduce more flexible variants of `mapId` and `mapComp`: for example, if `f` and `g` are composable morphisms and `fg` is such that `h : fg = f ≫ f`, we provide an isomorphism `F.mapComp' f g fg h : F.map fg ≅ F.map f ≫ F.map g`. We study the compatibilities of these isomorphisms with respect to composition with identities and associativity. Secondly, given a commutative square `t ≫ r = l ≫ b` in `B`, we construct an isomorphism `F.map t ≫ F.map r ≅ F.map l ≫ F.map b`. Co-authored-by: Christian Merten --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) maintainer-merge t-category-theory 168/0 Mathlib.lean,Mathlib/CategoryTheory/Bicategory/Functor/Pseudofunctor.lean,Mathlib/CategoryTheory/Bicategory/Functor/Strict.lean 3 17 ['callesonne', 'erdOne', 'github-actions', 'joelriou'] nobody
1-12557
1 day ago
1-78341
1 day ago
44-5911
44 days
25593 YaelDillies
author:YaelDillies
refactor(RelCat): use a type synonym for homs This improves automation and follows the new pattern for concrete categories (although `RelCat` is *not* a concrete category). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory 40/52 Mathlib/CategoryTheory/Category/RelCat.lean 1 10 ['YaelDillies', 'eric-wieser', 'github-actions'] nobody
1-10565
1 day ago
1-14706
1 day ago
1-14763
1 day
23555 Komyyy
author:Komyyy
feat(Mathlib/GroupTheory/SpecificGroups/Alternating): A_n is simple iff n = 3 or 5 ≤ n --- For reviewers: This PR is large. Please don't hesitate to let me know if you'd prefer it to be split. - [x] depends on: #25299 - [x] depends on: #25314 - [x] depends on: #25367 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-algebra
label:t-algebra$
300/31 Mathlib/Algebra/Group/End.lean,Mathlib/GroupTheory/SpecificGroups/Alternating.lean,Mathlib/GroupTheory/SpecificGroups/KleinFour.lean,Mathlib/GroupTheory/Subgroup/Simple.lean 4 11 ['AntoineChambert-Loir', 'Komyyy', 'acmepjz', 'ajirving', 'github-actions', 'mathlib4-dependent-issues-bot', 'tb65536'] nobody
1-10503
1 day ago
1-10503
1 day ago
3-21376
3 days
25587 YaelDillies
author:YaelDillies
refactor: make `Rel` less see-through There is tension throughout the library between considering relations between `α` and `β` simply as `α → β → Prop`, or as a bundled object `Rel α β` with dedicated operations and API. The former approach is used almost everywhere as it is very lightweight and has arguably native support from core Lean features, but it cracks at the seams whenever one starts talking about operations on relations. For example: * composition of relations `R : α → β → Prop`, `S : β → γ → Prop` is the unwieldy `Relation.Comp R S := fun a c ↦ ∃ b, R a b ∧ S b c` * map of a relation `R : α → β → Prop`, under `f : α → γ`, `g : β → δ` is the monstruous `Relation.map R f g := fun c d ↦ ∃ a b, r a b ∧ f a = c ∧ g b = d`. The latter approach is embodied by the existing type `Rel α β`, with dedicated notation like `○` for composition. It makes it much easier to reason about operations relations, but currently its API suffers from the leakage of its definition as ``` def Rel (α β : Type*) := α → β → Prop ``` The fact that `Rel` isn't an `abbrev` confuses automation. But simply making it an `abbrev` would kill the point of having a separate less see-through type to perform relation operations on. A final point, and the original motivation for this refactor, is that uniform spaces need a theory of relations on a type `α` as elements of `Set (α × α)`. This cannot be worked around, since `Set (α × α)` is the type of elements of a filter on `α × α`. This theory is already developed in `Topology.UniformSpace.Defs`, and duplicates the existing `Rel` material. This PR is a proposal to refactor `Rel` to be less see-through by redefining it as ``` abbrev Rel (α β : Type*) := Set (α × β) ``` This has several advantages: * The use of `α × β` means that one can't abuse the defeq of `Rel α β` with the function type `α → β → Prop`. * Instead, we get to provide an explicit notation `a ~[R] b` that very closely follows the paper convention `a ~R b` of using relations as infixes. This notation is scoped to the `Rel` namespace. * The use of `Set` is an extra layer of indirection to avoid automation confusing `Rel α β` with `α × β → Prop`. * It can directly be used in the theory of uniform spaces because of the syntactic equality between `Rel α α` and `Set (α × α)`. * A relation can still be defined from an explicit function `α → β → Prop`, with nice notation: What was previously `fun a b ↦ R a b` becomes `{(a, b) | R a b}`. * In general, fallout is manageably small and easily fixed by inserting the `{(a, b) | R a b}` and `a ~[R] b` notations. The benefits can be seen in places like `CategoryTheory.Category.RelCat` where automation is significantly improved, or `Combinatorics.Hall.Basic` where defeq abuse is avoided and dot notation becomes available. --- - [ ] depends on: #25593 I will add deprecations once CI passes and people agree this is a step forward. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data RFC blocked-by-other-PR 391/471 Mathlib/CategoryTheory/Category/RelCat.lean,Mathlib/Combinatorics/Hall/Basic.lean,Mathlib/Combinatorics/SimpleGraph/Basic.lean,Mathlib/Combinatorics/SimpleGraph/Path.lean,Mathlib/Combinatorics/SimpleGraph/Subgraph.lean,Mathlib/Data/PFun.lean,Mathlib/Data/Rel.lean,Mathlib/Order/Filter/Partial.lean,Mathlib/Order/JordanHolder.lean,Mathlib/Order/KrullDimension.lean,Mathlib/Order/Rel/GaloisConnection.lean,Mathlib/Order/RelSeries.lean,Mathlib/RingTheory/Ideal/AssociatedPrime/Finiteness.lean,Mathlib/RingTheory/Length.lean,Mathlib/RingTheory/Spectrum/Prime/LTSeries.lean 15 4 ['YaelDillies', 'eric-wieser', 'github-actions', 'mathlib4-dependent-issues-bot'] nobody
1-10160
1 day ago
1-13471
1 day ago
0-10145
2 hours
22834 joelriou
author:joelriou
feat(CategoryTheory): lifting properties and parametrized adjunctions Given a parametrized adjunction `adj₂ : F ⊣₂ G` between bifunctors `F : C₁ ⥤ C₂ ⥤ C₃` and `G : C₁ᵒᵖ ⥤ C₃ ⥤ C₂`, three maps `f₁ : X₁ ⟶ Y₁` in `C₁`, `f₂ : X₂ ⟶ Y₂` in `C₂`, and `f₃ : X₃ ⟶ Y₃` in `C₃`, this PR shows that `f₃` has the right lifting property with respect to the "inclusion" of the pushout of `(F.obj Y₁).obj X₂` and `(F.obj X₁).obj Y₂` along `(F.obj X₁).obj X₂` into `(F.obj Y₁).obj Y₂` if and only if `f₂` has the left lifting property with respect to the projection map from `(G.obj Y₁).obj X₃` to the pullback of `(G.obj (op X₁)).obj X₃` and `(G.obj (op Y₁)).obj Y₃` over `(G.obj (op X₁)).obj Y₃`. (In homotopical algebra, this is typically used for the adjunction between the tensor product and the internal hom.) --- - [x] depends on: #22828 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory 309/0 Mathlib.lean,Mathlib/CategoryTheory/LiftingProperties/Basic.lean,Mathlib/CategoryTheory/LiftingProperties/ParametrizedAdjunction.lean 3 10 ['github-actions', 'joelriou', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'robin-carlier'] nobody
1-9993
1 day ago
17-77605
17 days ago*
17-77596
17 days*
25596 Komyyy
author:Komyyy
feat: the Riemann zeta function is meromorphic (1/2) This PR just renames a file to make the git diff in PR #25597 cleaner. --- This PR renames the file `Analysis.Meromorphic.Gamma` to `Analysis.Meromorphic.Complex` without deprecating the original file, but I think this is fine since it was only added yesterday. - [ ] depends on: #25600 (#25600 isn't depended directly, but this PR shouldn't be merged before ready to merge #25597.) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) file-removed t-analysis blocked-by-other-PR 1/1 Mathlib.lean,Mathlib/Analysis/Meromorphic/Complex.lean 2 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
1-9056
1 day ago
1-9186
1 day ago
0-1463
24 minutes
25597 Komyyy
author:Komyyy
feat: the Riemann zeta function is meromorphic (2/2) Also proves that the Hurwitz zeta function is meromorphic. This PR is split from #25596 to leave a good git diff history. --- The PR #25596 renames the file `Analysis.Meromorphic.Gamma` to `Analysis.Meromorphic.Complex` without deprecating the original file, but I think this is fine since it was only added yesterday. For reviewers: It's welcome to merge master after #25596 is merged. - [ ] depends on: #25596 - [ ] depends on: #25600 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) file-removed t-analysis blocked-by-other-PR 72/23 Mathlib.lean,Mathlib/Analysis/Meromorphic/Complex.lean,Mathlib/Analysis/Meromorphic/Gamma.lean,Mathlib/Topology/ContinuousOn.lean 4 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
1-8406
1 day ago
1-9122
1 day ago
0-91
1 minute
24541 pfaffelh
author:pfaffelh
feat(Topology/Compactness/CompactSystem): introduce compact Systems A compact system is a set systems with the property that, whenever a countable intersections of sets in the set system is empty, there is a finite subset of sets with empty intersection. These are needed e.g. in measure theory if one wants to show sigma-additivity of a set function on a ring. * Main result: The set of sets which are either compact and closed, or `univ`, is a compact system. * Introduce `Dissipate s x := ⋂ y ≤ x, s y` (Data/Set/Dissipate), which is parallel to Data/Set/Accumulate. Co-authored-by: Rémy Degenne remydegenne@gmail.com new-contributor t-measure-probability 453/2 Mathlib.lean,Mathlib/Data/Set/Accumulate.lean,Mathlib/Data/Set/Dissipate.lean,Mathlib/MeasureTheory/PiSystem.lean,Mathlib/Topology/Compactness/CompactSystem.lean 5 74 ['github-actions', 'leanprover-community-bot-assistant', 'pfaffelh', 'sgouezel'] nobody
1-7437
1 day ago
1-7437
1 day ago
20-41251
20 days
25601 YaelDillies
author:YaelDillies
chore(CategoryTheory): unsimp `Mon_Class.tensorObj.one_def` This lemma loops with `IsMon_Hom.one_hom` applied to `(λ_ N.X).inv`, as evidenced by the following trace: ``` [Meta.Tactic.simp.rewrite] Mon_Class.tensorObj.one_def:1000: Mon_Class.one ==> (λ_ (𝟙_ C)).inv ≫ (Mon_Class.one ⊗ Mon_Class.one) [Meta.Tactic.simp.rewrite] id_tensorHom:1000: 𝟙 (𝟙_ C) ⊗ Mon_Class.one ==> 𝟙_ C ◁ Mon_Class.one [Meta.Tactic.simp.rewrite] id_whiskerLeft:1000: 𝟙_ C ◁ Mon_Class.one ==> (λ_ (𝟙_ C)).hom ≫ Mon_Class.one ≫ (λ_ N.X).inv [Meta.Tactic.simp.rewrite] IsMon_Hom.one_hom:1000: Mon_Class.one ≫ (λ_ N.X).inv ==> Mon_Class.one ``` Alternatively, `one_hom` is fine since it is the equivalent of `map_one` while `one_def` is not fine since it is the equivalent of `Algebra.TensorProduct.one_def`. Do the same thing for the `mul` lemmas and the `Mon_` versions. From Toric --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) toric t-category-theory easy 21/15 Mathlib/Algebra/Category/CoalgCat/ComonEquivalence.lean,Mathlib/CategoryTheory/Monoidal/Bimon_.lean,Mathlib/CategoryTheory/Monoidal/Hopf_.lean,Mathlib/CategoryTheory/Monoidal/Mon_.lean 4 1 ['github-actions'] nobody
1-7179
1 day ago
1-9269
1 day ago
1-9283
1 day
25333 fbarroero
author:fbarroero
Primitivity and `Ideal.span (p.coeffs.toSet)` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra WIP
label:t-algebra$
164/0 Mathlib.lean,Mathlib/Algebra/Polynomial/Basic.lean,Mathlib/RingTheory/Polynomial/ContentIdeal.lean 3 1 ['github-actions'] nobody
1-5630
1 day ago
9-15460
9 days ago
0-1263
21 minutes
25603 callesonne
author:callesonne
feat(Bicategory/InducedBicategory): add induced bicategories This PR adds a way of inducing a full bicategory structure on given type of objects with a map to the objects of some bicategory (i.e. with all 1-morphisms and all 2-morphisms). I have not tried to implement "locally induced bicategories" which should allow for a sub-class of 1-morphisms as well. This is because copying the naive approach and replacing the map `F` as for induced categories with a functor, one runs into issues when the equalities in `F.map_comp` and `F.map_id` are not defeq equalities. One could probably define locally full sub-bicategories using a pair of `ObjectProperty` + `MorphismProperty` to ensure that the inclusions are actually defeq, but I did not want to get into this. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory 68/0 Mathlib.lean,Mathlib/CategoryTheory/Bicategory/InducedBicategory.lean 2 1 ['github-actions'] nobody
1-2825
1 day ago
1-2893
1 day ago
1-2884
1 day
25604 sgouezel
author:sgouezel
feat: make sure that the simp normal form of equiv-like classes pushes `symm` and `trans` to the right This follows the usual convention for coercions. See discussion at [#mathlib4 > simp normal form for symm and coercions @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/simp.20normal.20form.20for.20symm.20and.20coercions/near/522879475) For each equiv class, after the PR we should have lemmas like ```lean @[simp] lemma coe_toEquiv (e : G ≃+c[a, b] H) : ⇑e.toEquiv = e := rfl @[simp] lemma coe_symm_toEquiv (e : G ≃+c[a, b] H) : ⇑e.toEquiv.symm = e.symm := rfl @[simp] lemma toEquiv_symm (e : G ≃+c[a, b] H) : e.symm.toEquiv = e.toEquiv.symm := rfl @[simp] lemma toEquiv_trans (e₁ : G ≃+c[a, b] H) (e₂ : H ≃+c[b, c] K) : (e₁.trans e₂).toEquiv = e₁.toEquiv.trans e₂.toEquiv := rfl ``` The PR does not complete this task, because it would require killing the coercion from EquivLike classes to Equivs (which I am planning to do in a subsequent PR), but it is a significant first step in this direction. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 196/64 Mathlib/Algebra/AddConstMap/Equiv.lean,Mathlib/Algebra/Algebra/Equiv.lean,Mathlib/Algebra/Module/Equiv/Basic.lean,Mathlib/Algebra/Module/Equiv/Defs.lean,Mathlib/Algebra/Module/ZLattice/Covolume.lean,Mathlib/Analysis/InnerProductSpace/PiL2.lean,Mathlib/Analysis/InnerProductSpace/TwoDim.lean,Mathlib/Analysis/Normed/Affine/Isometry.lean,Mathlib/Analysis/Normed/Affine/MazurUlam.lean,Mathlib/Analysis/Normed/Operator/Banach.lean,Mathlib/Analysis/Normed/Operator/LinearIsometry.lean,Mathlib/Analysis/NormedSpace/HahnBanach/Extension.lean,Mathlib/GroupTheory/Perm/Option.lean,Mathlib/LinearAlgebra/AffineSpace/AffineEquiv.lean,Mathlib/LinearAlgebra/AffineSpace/ContinuousAffineEquiv.lean,Mathlib/LinearAlgebra/RootSystem/IsValuedIn.lean,Mathlib/Logic/Equiv/Option.lean,Mathlib/MeasureTheory/Measure/Haar/InnerProductSpace.lean,Mathlib/MeasureTheory/Measure/Lebesgue/Complex.lean,Mathlib/ModelTheory/Algebra/Field/IsAlgClosed.lean,Mathlib/NumberTheory/NumberField/Discriminant/Defs.lean,Mathlib/Order/Hom/Basic.lean,Mathlib/Order/Hom/WithTopBot.lean,Mathlib/RingTheory/Bialgebra/Equiv.lean,Mathlib/RingTheory/Coalgebra/Equiv.lean,Mathlib/RingTheory/DedekindDomain/Different.lean,Mathlib/RingTheory/PowerBasis.lean,Mathlib/Topology/Algebra/Module/Equiv.lean,Mathlib/Topology/Algebra/Module/LinearPMap.lean,Mathlib/Topology/MetricSpace/DilationEquiv.lean,Mathlib/Topology/VectorBundle/Basic.lean 31 1 ['github-actions'] nobody
0-83506
23 hours ago
0-83506
23 hours ago
0-84326
23 hours
25602 DavidLedvinka
author:DavidLedvinka
feat(Probability): Law of the product of random variables Adds `IndepFun.map_mul_eq_map_mconv_map₀` and `IndepFun.map_mul_eq_map_mconv_map` which show that the law of the product of independent random variables is the convolution of their laws. Uses this to show that the sum of independent real gaussian variables is a real gaussian random variable. Also fix a notation change that I missed in #25434. t-measure-probability 33/2 Mathlib/MeasureTheory/Group/Convolution.lean,Mathlib/Probability/Distributions/Gaussian/Real.lean,Mathlib/Probability/Independence/Basic.lean 3 3 ['DavidLedvinka', 'Komyyy', 'github-actions'] nobody
0-83198
23 hours ago
1-8869
1 day ago
1-8854
1 day
23117 pfaffelh
author:pfaffelh
feat(MeasureTheory): finite unions of sets in a semi-ring (in terms of measure theory) form a ring : Finite unions of sets in a semi-ring (in terms of measure theory) form a ring The set containing finite unions of sets in a semi-ring are a ring. Part of `MeasureTheory.SetSemiring` is moved to the new file `MeasureTheory.SetRing`. --- - [ ] depends on: #22714 [contains changes in `SetSemiring` as well] large-import new-contributor t-measure-probability blocked-by-other-PR 453/104 Mathlib.lean,Mathlib/Data/Set/Lattice.lean,Mathlib/Data/Set/Pairwise/Lattice.lean,Mathlib/Data/Set/Prod.lean,Mathlib/MeasureTheory/MeasurableSpace/Pi.lean,Mathlib/MeasureTheory/Measure/AddContent.lean,Mathlib/MeasureTheory/PiSystem.lean,Mathlib/MeasureTheory/SetAlgebra.lean,Mathlib/MeasureTheory/SetRing.lean,Mathlib/MeasureTheory/SetSemiring.lean,lakefile.lean 11 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
0-82630
22 hours ago
1-2475
1 day ago
0-1301
21 minutes
25585 Paul-Lez
author:Paul-Lez
feat(Tactic/Linters/DeprecatedSimpLemma): lint for deprecated simp lemmas The deprecated simp lemma linter flags declarations that have both the `deprecated` and `simp` attributes. See Zulip discussion: [#mathlib4 > Help with Mathlib.Order.Interval.Finset.Defs @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Help.20with.20Mathlib.2EOrder.2EInterval.2EFinset.2EDefs/near/505994843) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-linter awaiting-author 105/0 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter/DeprecatedSimpLemma.lean,MathlibTest/DeprecatedSimpLemmaTest.lean 4 7 ['adomani', 'github-actions', 'grunweg'] nobody
0-81963
22 hours ago
0-81963
22 hours ago
0-34675
9 hours
25605 mans0954
author:mans0954
feature(RingTheory/Polynomial/SmallDegreeVieta): Polynomial versions of results in Algebra.QuadraticDiscriminant Provide `R[X]` versions of results about quadratic polynomials and their discriminants --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
57/0 Mathlib/RingTheory/Polynomial/SmallDegreeVieta.lean 1 2 ['github-actions', 'mans0954'] nobody
0-81404
22 hours ago
0-81404
22 hours ago
0-81395
22 hours
25582 grunweg
author:grunweg
fix/feat(PR_summary): improve messages about renamed and removed files We want to encourange adding module deprecations in a follow-up PR. Hence, - do not warn if such declarations are missing (but add an informational message, asking for a follow-up PR) - do warn if a deprecated_module attribute is present, and suggest a follow-up pull request instead. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 21/6 .github/workflows/PR_summary.yml 1 6 ['adomani', 'eric-wieser', 'github-actions', 'grunweg'] nobody
0-80175
22 hours ago
0-80376
22 hours ago
0-80419
22 hours
24542 pfaffelh
author:pfaffelh
feat (Topology/Compactness/CompactSystem): Closed and compact square cylinders form a compact system. feat (Topology/Compactness/CompactSystem): Closed and compact square cylinders form a compact system. A square cylinder is a set of the form `s.pi t` in a product space. A closed compact square cylinder has `IsClosed (t i)` and `IsCompact (t i)` for all `i ∈ s`. This set system is a compact system (as introduced in PR #24541). Streamline the definition of square cylinders in MeasureTheory/Constructions/Cylinders on the way. Co-authors: Rémy Degenne remy.degenne@inria.fr --- - [x] depends on: #24541 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-topology blocked-by-other-PR 264/66 Mathlib/Data/Set/Prod.lean,Mathlib/MeasureTheory/Constructions/Cylinders.lean,Mathlib/MeasureTheory/Constructions/ProjectiveFamilyContent.lean,Mathlib/Topology/Compactness/CompactSystem.lean 4 4 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
0-80012
22 hours ago
0-84878
23 hours ago
0-192
3 minutes
25600 Komyyy
author:Komyyy
refactor: lemma expressing `ContinuousAt` using a punctured neighbourhood --- This lemma is used to prove that the Riemann zeta function is meromorphic in #25597. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) maintainer-merge t-topology 4/0 Mathlib/Topology/ContinuousOn.lean 1 5 ['Komyyy', 'github-actions', 'grunweg'] nobody
0-79228
22 hours ago
0-79228
22 hours ago
1-4716
1 day
25190 wwylele
author:wwylele
feat(GroupTheory/Divisible): Add rational SMul and Module This is part of #25140. A torsion-free ℕ-divisible commutative group is a ℚ-module. This new instance could collide with existing instances such as ℚ-module on ℝ that comes from `Algebra`. I don't know how much an issue this is. I set the new instance with low priority so hopefully it won't interfere existing instances. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author 127/0 Mathlib/Data/Rat/Lemmas.lean,Mathlib/GroupTheory/Divisible.lean 2 2 ['eric-wieser', 'github-actions'] nobody
0-76373
21 hours ago
0-76373
21 hours ago
14-31640
14 days
25608 TOMILO87
author:TOMILO87
Add Beta distribution feat(Probability/Distributions): add Beta distribution Add the Beta distribution to the probability distributions in mathlib4. This implementation includes: - Definition of the Beta function over the reals - The probability density function (PDF) of the Beta distribution - Proof that the PDF integrates to 1 - Various lemmas about measurability and positivity properties The Beta distribution is a family of continuous probability distributions defined on the interval [0, 1] parametrized by two positive shape parameters, α and β, that control the shape of the distribution. The implementation follows a similar structure to other distributions in mathlib4, particularly the Gamma distribution, adapting the approach to the specific properties of the Beta distribution. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-measure-probability 257/0 Mathlib.lean,Mathlib/Probability/Distributions/Beta.lean 2 1 ['github-actions'] nobody
0-76007
21 hours ago
0-76019
21 hours ago
0-76075
21 hours
25573 JovanGerb
author:JovanGerb
feat: define `∃ x > y, ...` notation to mean `∃ x, y < x ∧ ...` This PR changes the elaboration of the binders `∃ x > y,` and `∀ x > y,` to use `<` instead of `>`, because we want to avoid working with `>` as much as possible (and similarly for `≥` vs `≤` ). The advantage is that we don't need to worry about rewriting with lemmas like `gt_iff_lt`. The disadvantage is that people might find this confusing. [#mathlib4 > naming convention for ≤ and < @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/naming.20convention.20for.20.E2.89.A4.20and.20.3C/near/522910464) The main changes are in `Mathlib.Init`, `Mathlib.Util.Delaborators` and `MathlibTest.delaborators`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta 59/52 Counterexamples/DiscreteTopologyNonDiscreteUniformity.lean,Mathlib/Algebra/Order/Monoid/Canonical/Defs.lean,Mathlib/Analysis/Analytic/Basic.lean,Mathlib/Analysis/BoxIntegral/Integrability.lean,Mathlib/Analysis/Calculus/UniformLimitsDeriv.lean,Mathlib/Analysis/Complex/Liouville.lean,Mathlib/Analysis/Complex/OpenMapping.lean,Mathlib/Analysis/Fourier/PoissonSummation.lean,Mathlib/Analysis/MellinTransform.lean,Mathlib/Analysis/Normed/Operator/Banach.lean,Mathlib/Dynamics/Ergodic/Conservative.lean,Mathlib/Dynamics/PeriodicPts/Defs.lean,Mathlib/Geometry/Manifold/IntegralCurve/ExistUnique.lean,Mathlib/Init.lean,Mathlib/MeasureTheory/Covering/LiminfLimsup.lean,Mathlib/MeasureTheory/Function/ConvergenceInMeasure.lean,Mathlib/MeasureTheory/Function/Egorov.lean,Mathlib/MeasureTheory/Function/StronglyMeasurable/Basic.lean,Mathlib/MeasureTheory/Integral/DivergenceTheorem.lean,Mathlib/MeasureTheory/Integral/Layercake.lean,Mathlib/NumberTheory/LSeries/SumCoeff.lean,Mathlib/Order/Filter/AtTopBot/Finite.lean,Mathlib/RingTheory/RootsOfUnity/PrimitiveRoots.lean,Mathlib/RingTheory/Valuation/Basic.lean,Mathlib/Topology/CWComplex/Classical/Finite.lean,Mathlib/Topology/ContinuousMap/Ideals.lean,Mathlib/Topology/EMetricSpace/Defs.lean,Mathlib/Topology/EMetricSpace/Paracompact.lean,Mathlib/Topology/LocallyFinite.lean,Mathlib/Topology/MetricSpace/Ultra/Basic.lean,Mathlib/Util/Delaborators.lean,MathlibTest/delaborators.lean 32 1 ['github-actions'] nobody
0-74524
20 hours ago
0-74636
20 hours ago
0-74625
20 hours
25348 wwylele
author:wwylele
feat(LinearAlgebra): add independent iSup to LinearPMap This is part of #25140. To obtain the Hahn embedding, we need to construct an partial linear map spanned by a family of submodules as the base case. This PR prepares for it. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-algebra
label:t-algebra$
94/2 Mathlib/LinearAlgebra/DFinsupp.lean,Mathlib/LinearAlgebra/LinearPMap.lean 2 2 ['eric-wieser', 'github-actions'] nobody
0-72911
20 hours ago
8-9468
8 days ago
8-9532
8 days
22603 pechersky
author:pechersky
chore(Topology): rename pi family from π to X Only in files that mentioned such a family, via a script: ``` git grep -e "π : . → Type" --name-only | rg Topology | xargs -I{} sed -i -e 's/π/X/g' {} ``` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) tech debt t-topology 238/238 Mathlib/Topology/AlexandrovDiscrete.lean,Mathlib/Topology/Algebra/InfiniteSum/Constructions.lean,Mathlib/Topology/Algebra/Module/Equiv.lean,Mathlib/Topology/Algebra/Order/LiminfLimsup.lean,Mathlib/Topology/Bases.lean,Mathlib/Topology/Bornology/Constructions.lean,Mathlib/Topology/Connected/Basic.lean,Mathlib/Topology/Connected/Clopen.lean,Mathlib/Topology/Connected/LocallyConnected.lean,Mathlib/Topology/Connected/TotallyDisconnected.lean,Mathlib/Topology/Constructions.lean,Mathlib/Topology/ContinuousOn.lean,Mathlib/Topology/EMetricSpace/Diam.lean,Mathlib/Topology/EMetricSpace/Pi.lean,Mathlib/Topology/ExtremallyDisconnected.lean,Mathlib/Topology/Inseparable.lean,Mathlib/Topology/MetricSpace/Basic.lean,Mathlib/Topology/MetricSpace/Infsep.lean,Mathlib/Topology/MetricSpace/ProperSpace.lean,Mathlib/Topology/MetricSpace/Pseudo/Pi.lean,Mathlib/Topology/Metrizable/Basic.lean,Mathlib/Topology/Order/Basic.lean,Mathlib/Topology/Separation/Hausdorff.lean,Mathlib/Topology/UniformSpace/Ascoli.lean 24 1 ['github-actions'] nobody
0-66274
18 hours ago
0-66296
18 hours ago
6-59911
6 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 awaiting-author 477/1 Mathlib.lean,Mathlib/Topology/MetricSpace/BundledFun.lean,Mathlib/Topology/UniformSpace/Ultra/Pseudometrizable.lean 3 7 ['ADedecker', 'fpvandoorn', 'github-actions', 'mathlib4-dependent-issues-bot', 'pechersky'] nobody
0-63809
17 hours ago
11-67758
11 days ago
15-31955
15 days
25009 mans0954
author:mans0954
feat(Analysis/SpecialFunctions/Trigonometric/Basic): sin and cos of multiples of π / 3 Add results: - `cos_ofNat_mul_pi_div_ofNat_of_eq_sub_one` : `cos ((n - 1) * π / n) = - cos π / n` - `cos_ofNat_mul_pi_div_ofNat_of_eq_two_mul_sub_one` : `cos ((2 * n - 1) * π / n) = cos π / n` - `cos_ofNat_mul_pi_div_ofNat_of_eq_add_one` : `cos ((n + 1) * π / n) = - cos π / n` And similar for `sin` and `tan`. This allows `norm_num` to prove results like: ``` example : cos (2 * π / 3) = - 1 / 2 := by norm_num example : cos (4 * π / 3) = - 1 / 2 := by norm_num example : cos (5 * π / 3) = 1 / 2 := by norm_num ``` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis 160/0 Mathlib/Algebra/Order/Monoid/NatCast.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Basic.lean,Mathlib/Data/Nat/Cast/Defs.lean,MathlibTest/trigonometry.lean 4 10 ['eric-wieser', 'github-actions', 'mans0954'] nobody
0-56185
15 hours ago
18-43609
18 days ago
20-38549
20 days
25515 jcommelin
author:jcommelin
chore: remove unneeded [nolint simpNF]s --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 48/77 Mathlib/Algebra/Group/Subsemigroup/Operations.lean,Mathlib/CategoryTheory/EqToHom.lean,Mathlib/CategoryTheory/Limits/Shapes/Biproducts.lean,Mathlib/CategoryTheory/Limits/Shapes/Products.lean,Mathlib/CategoryTheory/Subobject/Basic.lean,Mathlib/CategoryTheory/WithTerminal/Basic.lean,Mathlib/Data/Int/Cast/Basic.lean,Mathlib/Geometry/RingedSpace/Stalks.lean,Mathlib/LinearAlgebra/AffineSpace/AffineSubspace/Basic.lean,Mathlib/LinearAlgebra/Projection.lean,Mathlib/LinearAlgebra/TensorAlgebra/ToTensorPower.lean,Mathlib/MeasureTheory/Function/AEEqFun.lean,Mathlib/MeasureTheory/Function/SimpleFuncDense.lean,Mathlib/MeasureTheory/Integral/Bochner/Basic.lean,Mathlib/Topology/Sheaves/Stalks.lean,Mathlib/Topology/Specialization.lean 16 3 ['JovanGerb', 'github-actions'] nobody
0-55941
15 hours ago
0-56110
15 hours ago
2-7970
2 days
25304 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. - [ ] depends on: #25564 - [ ] depends on: #25562 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-analysis blocked-by-other-PR 333/0 Mathlib.lean,Mathlib/Analysis/Calculus/FDeriv/Partial.lean,Mathlib/Analysis/Normed/Operator/BoundedLinearMaps.lean,Mathlib/Topology/Algebra/Module/Equiv.lean 4 19 ['YaelDillies', 'github-actions', 'grunweg', 'igorkhavkine', 'mathlib4-dependent-issues-bot'] nobody
0-54140
15 hours ago
2-18241
2 days ago
4-14790
4 days
23676 Parcly-Taxel
author:Parcly-Taxel
chore: deprime `induction` for localizations and quotients All these removed instances of `induction'` generate only one subgoal. In some cases `obtain` can be used. The relevant instances were identified by adding the following to `Mathlib.Tactic.Cases` ```diff diff --git a/Mathlib/Tactic/Cases.lean b/Mathlib/Tactic/Cases.lean index 4a60db6c551..08c06520879 100644 --- a/Mathlib/Tactic/Cases.lean +++ b/Mathlib/Tactic/Cases.lean @@ -122,6 +122,16 @@ elab (name := induction') "induction' " tgts:(Parser.Tactic.elimTarget,+) g.assign result.elimApp let subgoals ← ElimApp.evalNames elimInfo result.alts withArg (generalized := fvarIds) (toClear := targetFVarIds) (toTag := toTag) + let body ← inferType targets[0]! + let names : Array Format := if withArg.1.getArgs.size > 1 then + (withArg.1.getArgs[1]!).getArgs.map Syntax.prettyPrint else Array.empty + let gens : Array Format := if genArg.1.getArgs.size > 1 then + (genArg.1.getArgs[1]!).getArgs.map Syntax.prettyPrint else Array.empty + let inductor : Format := if usingArg.1.getArgs.size > 1 then + Syntax.prettyPrint usingArg.1.getArgs[1]! else "~" + if subgoals.toList.length ≤ 1 then + logInfoAt tgts m!"{body.getAppFn.setPPExplicit true} {inductor} {gens} {names} \ + {subgoals.toList.length}" setGoals <| (subgoals ++ result.others).toList ++ gs /-- The `cases'` tactic is similar to the `cases` tactic in Lean 4 core, but the syntax for giving ``` and then examining [the output](https://github.com/leanprover-community/mathlib4/actions/runs/14270845291/job/40003467676). tech debt 71/77 Mathlib/Algebra/Module/LocalizedModule/Basic.lean,Mathlib/Algebra/Pointwise/Stabilizer.lean,Mathlib/Analysis/SpecialFunctions/Complex/Circle.lean,Mathlib/Analysis/SpecialFunctions/Pow/NNReal.lean,Mathlib/CategoryTheory/Action/Concrete.lean,Mathlib/CategoryTheory/Galois/EssSurj.lean,Mathlib/CategoryTheory/Limits/Types/Colimits.lean,Mathlib/CategoryTheory/Subobject/Basic.lean,Mathlib/CategoryTheory/Subobject/FactorThru.lean,Mathlib/CategoryTheory/Subobject/Lattice.lean,Mathlib/Data/Finset/NoncommProd.lean,Mathlib/Data/Finsupp/BigOperators.lean,Mathlib/Data/Fintype/Quotient.lean,Mathlib/Data/List/Cycle.lean,Mathlib/Data/Nat/ChineseRemainder.lean,Mathlib/Data/Setoid/Partition.lean,Mathlib/GroupTheory/Perm/Sign.lean,Mathlib/RingTheory/OreLocalization/Basic.lean,Mathlib/RingTheory/OreLocalization/Ring.lean 19 11 ['Parcly-Taxel', 'apnelson1', 'eric-wieser', 'github-actions', 'grunweg', 'leanprover-community-bot-assistant', 'urkud'] nobody
0-51824
14 hours ago
2-794
2 days ago
63-65172
63 days
25564 igorkhavkine
author:igorkhavkine
feat(Topology/Algebra/Module): interaction between ContinuousLinearMap.coprod and ContinuousLinearEquiv.prodComm `ContinuousLinearMap.coprod_comp_prodComm` shows that pre-composition of a coproduct with prodComm (swap) swaps the terms in the coproduct. A dependency of #25304. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis 7/0 Mathlib/Topology/Algebra/Module/Equiv.lean 1 12 ['YaelDillies', 'github-actions', 'grunweg', 'igorkhavkine'] nobody
0-51114
14 hours ago
0-51114
14 hours ago
0-69628
19 hours
25616 erdOne
author:erdOne
feat(RingTheory/Invariant): residue field extension is finite --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
51/0 Mathlib/FieldTheory/Galois/Basic.lean,Mathlib/RingTheory/Invariant/Basic.lean 2 1 ['github-actions'] nobody
0-47164
13 hours ago
0-47174
13 hours ago
0-47226
13 hours
24692 ScottCarnahan
author:ScottCarnahan
feat (RingTheory/HahnSeries/Basic): isomorphism of Hahn series induced by order isomorphism This PR introduces an isomorphism of Hahn series induced by an order isomorphism on the exponent posets. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order WIP 35/0 Mathlib/RingTheory/HahnSeries/Basic.lean 1 1 ['github-actions'] nobody
0-46897
13 hours ago
0-46897
13 hours ago
31-47622
31 days
25035 ScottCarnahan
author:ScottCarnahan
feat (Algebra/Module/Equiv/Defs): Linear equivalence between linear hom and semilinear hom. Given a ring homomorphism `σ₂ : R →+* R₂`, an `R`-module `M`, and a module `M₂` for both `R` and `R₂` satisfying `SMulCommClass R R₂ M₂` and `(σ₂ r) • x = r • x`, we produce an `R₂`-linear equivalence between `M →ₗ[R] M₂` and `M →ₛₗ[σ₂] M₂`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra WIP
label:t-algebra$
21/0 Mathlib/Algebra/Module/Equiv/Defs.lean 1 1 ['github-actions'] nobody
0-46884
13 hours ago
0-46884
13 hours ago
20-7584
20 days
25034 ScottCarnahan
author:ScottCarnahan
feat (Algebra/Module/Equiv/Basic): Restriction of scalars from a semilinear equivalence to a linear equivalence. If `M` and `M₂` are both `R`-modules and modules for `S` and `S₂`, respectively, then for any ring isomorphism `e` between `S` and `S₂` and any `e`-semilinear equivalence between `M` and `M₂` that respects the `R`-action, we obtain an `R`-linear equivalence between `M` and `M₂`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra WIP
label:t-algebra$
28/0 Mathlib/Algebra/Module/Equiv/Basic.lean 1 1 ['github-actions'] nobody
0-46859
13 hours ago
0-46859
13 hours ago
20-11468
20 days
25470 mans0954
author:mans0954
Low order roots of unity Compute some low order roots of unity. [Zulip discussion](https://leanprover.zulipchat.com/#narrow/channel/116395-maths/topic/roots.20of.20unity.20-.20computing.20low.20degree/with/520523576) Cubic case contributed by @MichaelStollBayreuth See also: #25215, #24828 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
182/0 Mathlib/Algebra/CharP/Invertible.lean,Mathlib/RingTheory/RootsOfUnity/Complex.lean 2 1 ['github-actions'] nobody
0-46136
12 hours ago
0-46136
12 hours ago
2-75320
2 days
24498 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`. --- Is there a better way to express `eq_toFun`? [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
33/13 Mathlib/RingTheory/HahnSeries/HEval.lean 1 2 ['github-actions', 'leanprover-community-bot-assistant'] nobody
0-45683
12 hours ago
0-45719
12 hours ago
37-42657
37 days
23849 chrisflav
author:chrisflav
feat(Data/Set): add `Set.encard_iUnion` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data 65/0 Mathlib/Algebra/BigOperators/Finprod.lean,Mathlib/Data/Set/Card/Arithmetic.lean,Mathlib/Data/Set/Finite/Lattice.lean 3 11 ['YaelDillies', 'chrisflav', 'github-actions'] YaelDillies
assignee:YaelDillies
0-42428
11 hours ago
31-25784
1 month ago
61-54575
61 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$
92/1 Mathlib.lean,Mathlib/Algebra/Ring/Equiv.lean,Mathlib/RingTheory/RingHom/FaithfullyFlat.lean,Mathlib/RingTheory/RingHom/Flat.lean 4 4 ['chrisflav', 'erdOne', 'github-actions', 'mathlib4-dependent-issues-bot'] nobody
0-42212
11 hours ago
30-36220
30 days ago
30-37286
30 days
24102 ScottCarnahan
author:ScottCarnahan
feat (RingTheory/HahnSeries): Powers of a binomial This PR introduces powers of a binomial `single g 1 - single g' 1` in a Hahn series, where the powers take values in a binomial ring. These series behave as one would expect with respect to addition of powers, and comparison with natural number powers. They are often used in the theory of vertex algebras. --- - [x] depends on: #24498 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra blocked-by-other-PR
label:t-algebra$
180/23 Mathlib.lean,Mathlib/RingTheory/HahnSeries/Addition.lean,Mathlib/RingTheory/HahnSeries/Binomial.lean,Mathlib/RingTheory/HahnSeries/HEval.lean,Mathlib/RingTheory/HahnSeries/Multiplication.lean,Mathlib/RingTheory/PowerSeries/Binomial.lean 6 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
0-41062
11 hours ago
0-41079
11 hours ago
15-33856
15 days
21740 101damnations
author:101damnations
feat(RepresentationTheory/Homological/GroupHomology/Basic): define group homology Let `k` be a commutative ring and `G` a group. This PR defines the group homology of `A : Rep k G` to be the homology of the complex $$\dots \to \bigoplus_{G^2} A \to \bigoplus_{G^1} A \to \bigoplus_{G^0} A$$ (using `Finsupp` for the objects) with differential $d_n$ sending $a\cdot (g_0, \dots, g_n)$ to $$\rho(g_0^{-1})(a)\cdot (g_1, \dots, g_n) + \sum_{i = 0}^{n - 1}(-1)^{i + 1}a\cdot (g_0, \dots, g_ig_{i + 1}, \dots, g_n) + (-1)^{n + 1}a\cdot (g_0, \dots, g_{n - 1})$$ (where `ρ` is the representation attached to `A`). We have a `k`-linear isomorphism $\bigoplus_{G^n} A \cong (A \otimes_k \left(\bigoplus_{G^n} k[G]\right))_G$ given by `Rep.coinvariantsTensorFreeLEquiv`. If we conjugate the `n`th differential in $(A \otimes_k P)_G$ by this isomorphism, where `P` is the bar resolution of `k` as a trivial `k`-linear `G`-representation, then the resulting map agrees with the differential $d_n$ defined above, a fact we prove. Hence our $d_n$ squares to zero, and we get $\mathrm{H}_n(G, A) \cong \mathrm{Tor}_n(A, k),$ where $\mathrm{Tor}$ is defined by deriving the second argument of the functor $(A, B) \mapsto (A \otimes_k B)_G.$ --- - [x] depends on: #21652 - [x] depends on: #21732 - [x] depends on: #21733 - [x] depends on: #21735 - [x] depends on: #21736 - [x] depends on: #21738 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) file-removed t-algebra
label:t-algebra$
236/17 Mathlib.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/Basic.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/Functoriality.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/Hilbert90.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/LowDegree.lean,Mathlib/RepresentationTheory/Homological/GroupHomology/Basic.lean,Mathlib/RepresentationTheory/Homological/Resolution.lean 7 n/a ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
0-41000
11 hours ago
unknown
unknown
13611 callesonne
author:callesonne
feat(FiberedCategory/HasFibers): define HasFibers class We define a class `HasFibers p` for a given functor `p : 𝒳 ⥤ 𝒮`. The point of this is to give the user the option to supply their own fiber categories, as often the standard fibers will not be definitionally the same as the (equivalent) categories one is interested in. Co-authored-by: Paul Lezeau --- This is the final PR in a sequence of PRs developing the theory of fibered categories that I will make for now. I will wait for the reviewing to catch up before I start working on more of these again, so as to not create too big of a backlog. - [x] depends on: #13603 - [x] depends on: #12982 - [x] depends on: #13416 - [x] depends on: #13410 - [x] depends on: #13393 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory 276/21 Mathlib.lean,Mathlib/CategoryTheory/FiberedCategory/Cartesian.lean,Mathlib/CategoryTheory/FiberedCategory/HasFibers.lean,Mathlib/CategoryTheory/FiberedCategory/HomLift.lean 4 26 ['callesonne', 'github-actions', 'joelriou', 'mathlib4-dependent-issues-bot'] nobody
0-40081
11 hours ago
233-21757
7 months ago*
0-571
9 minutes*
23339 joelriou
author:joelriou
feat(CategoryTheory): the colimit type of a functor to types Given a category `J` (with `J : Type u` and `[Category.{v} J]`) and a functor `F : J ⥤ Type w`, we introduce a type `F.ColimitType : Type (max u w)`, which satisfies a certain universal property of the colimit: it is defined as a suitable quotient of `Σ j, F.obj j`. This universal property is not expressed in a categorical way (as in general `Type (max u w)` is not the same as `Type u`). (This type `F.ColimitType` is basically the same as `CategoryTheory.Limits.Types.Quot` that is defined in `CategoryTheory.Limits.Types`, but we expand the API (with minimal imports to category theory) so that it may be used in future PRs to refactor both `DirectedSystem` and the construction of colimits in `Type`.) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory 273/0 Mathlib.lean,Mathlib/CategoryTheory/Limits/Types/ColimitType.lean 2 10 ['AntoineChambert-Loir', 'adamtopaz', 'erdOne', 'github-actions', 'joelriou'] adamtopaz
assignee:adamtopaz
0-39795
11 hours ago
0-39795
11 hours ago
53-13313
53 days
24794 chrisflav
author:chrisflav
feat(RingTheory/Presentation): core of a presentation If `P` is a presentation of `S` as an `R`-algebra and `R₀` a subring of `R` containing the coefficients of the relations of `P`, then there exists an `R₀`-algebra `S₀` such that `S` is isomorphic to the base change of `S₀` to `R`. This is a tool to remove Noetherian hypothesis in certain situations. --- - [x] depends on: #24788 - [x] depends on: #24786 - [x] depends on: #24785 [![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 4 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
0-39504
10 hours ago
0-42200
11 hours ago
0-43141
11 hours
24520 chrisflav
author:chrisflav
feat(Algebra/Pi): add various `AlgEquiv`s and `RingEquiv`s Add - `RingEquiv.sumArrowEquivProdArrow`: ring version of `Equiv.sumArrowEquivProdArrow`. - `AlgEquiv.sumArrowEquivProdArrow`: algebra version of `Equiv.sumArrowEquivProdArrow`. - `AlgEquiv.piCongrLeft'`: algebra version of `Equiv.piCongrLeft`. - `AlgEquiv.piCongrLeft`: algebra version of `Equiv.piCongrLeft`. - `AlgEquiv.funUnique`: algebra version of `Equiv.funUnique`. - `AlgEquiv.prodCongr`: algebra version of `Equiv.prodCongr`. The four last ones already have ring versions. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
116/1 Mathlib/Algebra/Algebra/Pi.lean,Mathlib/Algebra/Algebra/Prod.lean,Mathlib/Algebra/Ring/Equiv.lean 3 20 ['Ruben-VandeVelde', 'chrisflav', 'eric-wieser', 'github-actions', 'mistarro'] eric-wieser
assignee:eric-wieser
0-38754
10 hours ago
15-76048
15 days ago
39-8351
39 days
24379 chrisflav
author:chrisflav
feat(Algebra/AlgHom): `Unique` if target is `Subsingleton` --- [![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/Algebra/Equiv.lean,Mathlib/Algebra/Algebra/Hom.lean 2 6 ['chrisflav', 'eric-wieser', 'github-actions'] nobody
0-38535
10 hours ago
39-28735
1 month ago
39-64672
39 days
22714 pfaffelh
author:pfaffelh
feat: The finite product of semi-rings (in terms of measure theory) is a semi-ring. ~~Move results for rings (in terms of measure theory) to a separate file; was in Semiring.lean before.~~ For `∀ i ∈ s, IsSetSemiring (C i))`, the product `s.pi '' s.pi C` is a semiring. Prove two auxiliary lemmas in `Data.Set.Prod` needed on the way. large-import new-contributor t-measure-probability 264/14 Mathlib/Data/Set/Pairwise/Lattice.lean,Mathlib/Data/Set/Prod.lean,Mathlib/MeasureTheory/MeasurableSpace/Pi.lean,Mathlib/MeasureTheory/PiSystem.lean,Mathlib/MeasureTheory/SetSemiring.lean,lakefile.lean 6 15 ['EtienneC30', 'Paul-Lez', 'github-actions', 'leanprover-community-bot-assistant', 'pfaffelh', 'sgouezel'] EtienneC30
assignee:EtienneC30
0-38025
10 hours ago
0-38025
10 hours ago
23-54117
23 days
25442 oliver-butterley
author:oliver-butterley
feat(MeasureTheory.VectorMeasure) : add a definition of total variation for VectorMeasure This PR adds variation for any `VectorMeasure` using a supremum definition. Currently mathlib has `TotalVariation` defined for a signed measure using the Hahn-Jordan decomposition, but this doesn't generalise. Includes the result showing that for `SignedMeasure`s the two definitions coincide. Motivation: generally this is an important concept but specifically as a step for proving RMK in the complex case which in turn is a step to prove the spectral theorem. Co-authored-by: @yoh-tanimoto --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor RFC 664/0 Mathlib.lean,Mathlib/MeasureTheory/VectorMeasure/Variation.lean 2 4 ['github-actions', 'grunweg', 'oliver-butterley'] nobody
0-37769
10 hours ago
0-38103
10 hours ago
0-38511
10 hours
25050 linesthatinterlace
author:linesthatinterlace
feat: Add `Vector`/`List.Vector` equivalence Adds an equivalence between `Vector` and `List.Vector`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data 125/17 Mathlib/Data/Vector/Basic.lean,Mathlib/Data/Vector/Defs.lean,Mathlib/Logic/Equiv/Array.lean 3 57 ['digama0', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'linesthatinterlace'] nobody
0-37494
10 hours ago
0-40379
11 hours ago
6-55239
6 days
24430 RemyDegenne
author:RemyDegenne
feat(Probability): Fernique's theorem - invariance by rotation of Gaussian measures - Fernique's theorem - Corollary: the identity is in Lp for all finite p --- - [x] depends on: #24975 - [x] depends on: #24969 - [x] depends on: #24930 - [x] depends on: #24925 - [x] depends on: #24900 - [ ] depends on: #25532 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-measure-probability WIP 967/9 Mathlib.lean,Mathlib/MeasureTheory/Group/Convolution.lean,Mathlib/MeasureTheory/Measure/CharacteristicFunction.lean,Mathlib/Probability/Distributions/Fernique.lean,Mathlib/Probability/Distributions/Gaussian/Basic.lean,Mathlib/Probability/Distributions/Gaussian/Fernique.lean 6 9 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
0-37068
10 hours ago
0-37071
10 hours ago
0-0
0 seconds
25599 adomani
author:adomani
test: autolabel from forks --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) test-ci awaiting-author WIP 1/1 Mathlib/Tactic/Eval.lean,newFileOnMaster.md 2 3 ['adomani', 'bryangingechen', 'github-actions'] nobody
0-33809
9 hours ago
1-9271
1 day ago
0-0
0 seconds
24506 robin-carlier
author:robin-carlier
feat(Tactic/CategoryTheory): Initial lemmas for the `rotate_iso` tactic This PR records an initial set of lemmas to be used by the WIP `rotate_isos` tactic. --- - [ ] depends on: #24452 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta blocked-by-other-PR 496/0 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/CategoryTheory/RotateIsos/Cancelable.lean,Mathlib/Tactic/CategoryTheory/RotateIsos/Lemmas.lean,scripts/noshake.json 5 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
0-32763
9 hours ago
39-28930
1 month ago
0-47
47 seconds
25617 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 88/79 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/Synonym.lean 14 1 ['github-actions'] nobody
0-32126
8 hours ago
0-42925
11 hours ago
0-42910
11 hours
22790 mhk119
author:mhk119
feat: Extend `taylor_mean_remainder_lagrange` to `x < x_0` The `taylor_mean_remainder_lagrange` theorem has the assumption that $x_0 < x$. In many applications, we need $x < x_0$ and one cannot use the current version to obtain this (see [zulip](https://leanprover.zulipchat.com/#narrow/channel/116395-maths/topic/Taylor's.20theorem)). This PR introduces a set of theorems that push negations through Taylor expansions so that one can extend `taylor_mean_remainder_lagrange` to the case when $x < x_0$. These theorems should also be useful elsewhere since they are quite general. new-contributor t-analysis awaiting-author 393527/62 Mathlib/Algebra/Group/Equiv/Basic.lean,Mathlib/Algebra/Group/Hom/Basic.lean,Mathlib/Algebra/Group/Hom/Defs.lean,Mathlib/Algebra/Group/Subgroup/Basic.lean,Mathlib/Analysis/Calculus/Deriv/Basic.lean,Mathlib/Analysis/Calculus/IteratedDeriv/Lemmas.lean,Mathlib/Analysis/Calculus/Taylor.lean,README.md,build/ir/Mathlib/Algebra/Abs.c,build/ir/Mathlib/Control/Basic.c,build/ir/Mathlib/Control/Functor.c,build/ir/Mathlib/Control/SimpSet.c,build/ir/Mathlib/Data/Array/Defs.c,build/ir/Mathlib/Data/Bracket.c,build/ir/Mathlib/Data/HashMap.c,build/ir/Mathlib/Data/KVMap.c,build/ir/Mathlib/Data/Rat/Init.c,build/ir/Mathlib/Data/String/Defs.c,build/ir/Mathlib/Init/Algebra/Classes.c,build/ir/Mathlib/Init/CcLemmas.c,build/ir/Mathlib/Init/Control/Combinators.c,build/ir/Mathlib/Init/Core.c,build/ir/Mathlib/Init/Data/Bool/Basic.c,build/ir/Mathlib/Init/Data/Fin/Basic.c,build/ir/Mathlib/Init/Data/Int/Basic.c,build/ir/Mathlib/Init/Data/List/Basic.c,build/ir/Mathlib/Init/Data/Nat/Basic.c,build/ir/Mathlib/Init/Data/Nat/Notation.c,build/ir/Mathlib/Init/Data/Ordering/Basic.c,build/ir/Mathlib/Init/Data/Prod.c,build/ir/Mathlib/Init/Data/Quot.c,build/ir/Mathlib/Init/Data/Sigma/Basic.c,build/ir/Mathlib/Init/Function.c,build/ir/Mathlib/Init/Logic.c,build/ir/Mathlib/Init/Propext.c,build/ir/Mathlib/Init/Quot.c,build/ir/Mathlib/Init/Set.c,build/ir/Mathlib/Init/ZeroOne.c,build/ir/Mathlib/Lean/CoreM.c,build/ir/Mathlib/Lean/Elab/Tactic/Basic.c,build/ir/Mathlib/Lean/EnvExtension.c,build/ir/Mathlib/Lean/Exception.c,build/ir/Mathlib/Lean/Expr.c,build/ir/Mathlib/Lean/Expr/Basic.c,build/ir/Mathlib/Lean/Expr/ReplaceRec.c,build/ir/Mathlib/Lean/Expr/Traverse.c,build/ir/Mathlib/Lean/Linter.c,build/ir/Mathlib/Lean/LocalContext.c,build/ir/Mathlib/Lean/Message.c,build/ir/Mathlib/Lean/Meta.c,build/ir/Mathlib/Lean/Meta/Basic.c,build/ir/Mathlib/Lean/Meta/DiscrTree.c,build/ir/Mathlib/Lean/Meta/Simp.c,build/ir/Mathlib/Mathport/Attributes.c,build/ir/Mathlib/Mathport/Notation.c,build/ir/Mathlib/Mathport/Rename.c,build/ir/Mathlib/Tactic/Alias.c,build/ir/Mathlib/Tactic/ApplyCongr.c,build/ir/Mathlib/Tactic/ApplyWith.c,build/ir/Mathlib/Tactic/Basic.c,build/ir/Mathlib/Tactic/Cases.c,build/ir/Mathlib/Tactic/CasesM.c,build/ir/Mathlib/Tactic/Classical.c,build/ir/Mathlib/Tactic/Clear!.c,build/ir/Mathlib/Tactic/ClearExcept.c,build/ir/Mathlib/Tactic/Clear_.c,build/ir/Mathlib/Tactic/Coe.c,build/ir/Mathlib/Tactic/Congr!.c,build/ir/Mathlib/Tactic/Constructor.c,build/ir/Mathlib/Tactic/Conv.c,build/ir/Mathlib/Tactic/Convert.c,build/ir/Mathlib/Tactic/Core.c,build/ir/Mathlib/Tactic/Eqns.c,build/ir/Mathlib/Tactic/Existsi.c,build/ir/Mathlib/Tactic/FailIfNoProgress.c,build/ir/Mathlib/Tactic/GeneralizeProofs.c,build/ir/Mathlib/Tactic/GuardGoalNums.c,build/ir/Mathlib/Tactic/GuardHypNums.c,build/ir/Mathlib/Tactic/Have.c,build/ir/Mathlib/Tactic/HelpCmd.c,build/ir/Mathlib/Tactic/HigherOrder.c,build/ir/Mathlib/Tactic/InferParam.c,build/ir/Mathlib/Tactic/Inhabit.c,build/ir/Mathlib/Tactic/LabelAttr.c,build/ir/Mathlib/Tactic/LeftRight.c,build/ir/Mathlib/Tactic/MkIffOfInductiveProp.c,build/ir/Mathlib/Tactic/Monotonicity/Attr.c,build/ir/Mathlib/Tactic/NthRewrite.c,build/ir/Mathlib/Tactic/PermuteGoals.c,build/ir/Mathlib/Tactic/PrintPrefix.c,build/ir/Mathlib/Tactic/ProjectionNotation.c,build/ir/Mathlib/Tactic/RSuffices.c,build/ir/Mathlib/Tactic/Relation/Rfl.c,build/ir/Mathlib/Tactic/Relation/Symm.c,build/ir/Mathlib/Tactic/Relation/Trans.c,build/ir/Mathlib/Tactic/Rename.c,build/ir/Mathlib/Tactic/RenameBVar.c,build/ir/Mathlib/Tactic/Replace.c,build/ir/Mathlib/Tactic/RunCmd.c,build/ir/Mathlib/Tactic/ScopedNS.c 492 11 ['Paul-Lez', 'github-actions', 'grunweg'] nobody
0-30324
8 hours ago
60-27268
1 month ago
30-77130
30 days
25308 pechersky
author:pechersky
chore(Algebra/Ring/Subring): simp tag `Subring.smul_def` --- [![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. t-algebra awaiting-author
label:t-algebra$
7/3 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/Ring/Subring/Basic.lean,Mathlib/Algebra/Ring/Subsemiring/Basic.lean,Mathlib/RingTheory/OreLocalization/Basic.lean 7 2 ['eric-wieser', 'github-actions'] nobody
0-28572
7 hours ago
10-24448
10 days ago
0-24882
6 hours
24628 pechersky
author:pechersky
feat(Topology/UniformSpace/Ultra): completion is ultra uniformity iff base is --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology 162/7 Mathlib.lean,Mathlib/Order/Filter/Map.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 8 11 ['ADedecker', 'D-Thomine', 'github-actions'] nobody
0-28560
7 hours ago
0-28560
7 hours ago
3-50967
3 days
25621 joelriou
author:joelriou
refactor(CategoryTheory/Limits): generalize universes for colimits of representables --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory WIP 756/21 Mathlib.lean,Mathlib/AlgebraicTopology/SingularSet.lean,Mathlib/CategoryTheory/Elements.lean,Mathlib/CategoryTheory/Limits/PresheafULift.lean,Mathlib/CategoryTheory/Types.lean,Mathlib/CategoryTheory/Yoneda.lean 6 1 ['github-actions'] nobody
0-27344
7 hours ago
0-27425
7 hours ago
0-1
1 second
25458 ADedecker
author:ADedecker
feat: integrability assuming that the domain/codomain is a subsingleton I really only care about the codomain being trivial for #25455 , but thought I'd add some more lemmas on the way. The `@[simp]` attributes are here to make sure that these lemmas are accessible to the `nontriviality` tactic. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-measure-probability awaiting-author 35/0 Mathlib/MeasureTheory/Function/L1Space/HasFiniteIntegral.lean,Mathlib/MeasureTheory/Function/L1Space/Integrable.lean,Mathlib/MeasureTheory/Integral/IntegrableOn.lean 3 6 ['ADedecker', 'Ruben-VandeVelde', 'github-actions', 'leanprover-bot', 'sgouezel'] nobody
0-27059
7 hours ago
0-27059
7 hours ago
4-54473
4 days
24452 robin-carlier
author:robin-carlier
feat(Tactic/CategoryTheory): `Cancelable` boilerplate for the `rotate_isos` WIP tactic This PR adds some boilerplate that will be used in a forthcoming PR implementing a `rotate_isos` tactic that aims to provide easy ways of moving one or more morphisms that can be inferred to be isomorphisms (not necessarily through the `IsIso typeclass, but also directly by recognizing them as e.g components of natural isomorphisms, or functor application to such morphisms). The boilerplate in this PR abstracts the notion of a cancelable expression for a morphism in a composition of (iso)morphisms in a category, and records a global reference to a list of "cancelable factories", _i.e_ functions that try to recognize term in an expression as a "cancelable" morphism, and provides helper to register such functions. --- First part of a series of 3 PRs contributing the `rotate_isos` tactic to mathlib. Second part will actually implement the tactic, and provide a test suite. Please read the description of the second PR (#24454) to get more details. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory t-meta awaiting-author 162/0 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/CategoryTheory/RotateIsos/Cancelable.lean,scripts/noshake.json 4 8 ['callesonne', 'github-actions', 'robin-carlier'] nobody
0-26112
7 hours ago
0-84530
23 hours ago
38-38748
38 days
25230 Thmoas-Guan
author:Thmoas-Guan
feat(Algebra): definition of cohen macaulay In this PR, we added the definition of CM module, CM local ring (extending local ring), and CM ring. We also proved Theorem 30, Chater 6, _Commutative Algebra_, Matsumura. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import 2211/37 Mathlib.lean,Mathlib/Algebra/Category/Grp/Preadditive.lean,Mathlib/Algebra/Homology/ExactSequence.lean,Mathlib/Algebra/Module/Submodule/Lattice.lean,Mathlib/LinearAlgebra/Quotient/Basic.lean,Mathlib/RingTheory/CohenMacaulay/Basic.lean,Mathlib/RingTheory/Ideal/AssociatedPrime/Localization.lean,Mathlib/RingTheory/Ideal/MinimalPrime/Localization.lean,Mathlib/RingTheory/KrullDimension/Module.lean,Mathlib/RingTheory/KrullDimension/Regular.lean,Mathlib/RingTheory/Nakayama.lean,Mathlib/RingTheory/Regular/Category.lean,Mathlib/RingTheory/Regular/Depth.lean,Mathlib/RingTheory/Regular/Ischebeck.lean,Mathlib/RingTheory/Spectrum/Prime/LTSeries.lean,Mathlib/RingTheory/Support.lean 16 n/a ['github-actions', 'leanprover-community-bot-assistant'] nobody
0-25003
6 hours ago
unknown
unknown
25334 matthewjasper
author:matthewjasper
feat(RingTheory/Flat): Add theorems relating Submodule.torsion and Module.Flat Co-authored-by: Kevin Buzzard --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) FLT new-contributor t-algebra
label:t-algebra$
202/0 Mathlib.lean,Mathlib/Algebra/Algebra/Bilinear.lean,Mathlib/Algebra/Module/LocalizedModule/Basic.lean,Mathlib/RingTheory/Flat/TorsionFree.lean,Mathlib/RingTheory/Ideal/IsPrincipal.lean 5 13 ['alreadydone', 'erdOne', 'github-actions', 'kbuzzard'] nobody
0-24330
6 hours ago
9-7627
9 days ago
9-7626
9 days
22420 pechersky
author:pechersky
feat(Order/Prod/Lex/{Hom,Monoid,GroupWithZero}): ordered inclusions and projections of prod of ordered groups --- - [x] depends on: #22402 - [x] depends on: #25466 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order t-algebra
label:t-algebra$
363/0 Mathlib.lean,Mathlib/Algebra/GroupWithZero/WithZero.lean,Mathlib/Algebra/Order/GroupWithZero/Canonical.lean,Mathlib/Algebra/Order/Hom/Monoid.lean,Mathlib/Order/Prod/Lex/GroupWithZero.lean,Mathlib/Order/Prod/Lex/Hom.lean,Mathlib/Order/Prod/Lex/Monoid.lean 7 17 ['YaelDillies', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'pechersky'] YaelDillies
assignee:YaelDillies
0-23974
6 hours ago
0-23981
6 hours ago
58-17922
58 days
25562 igorkhavkine
author:igorkhavkine
feat(Analysis/Normed/Operator): continuity of forming `ContinuousLinearMap` coproducts pointwise `Continuous(|On).clm_coprod` shows that the pointwise coproduct of two continuous functions valued in ContinuousLinearMap is itself continuous. A dependency of #25304. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis 16/0 Mathlib/Analysis/Normed/Operator/BoundedLinearMaps.lean 1 4 ['YaelDillies', 'github-actions', 'igorkhavkine'] nobody
0-22777
6 hours ago
0-55896
15 hours ago
0-74699
20 hours
25623 mattrobball
author:mattrobball
feat: decidable equality for `Quiver.Path` Given a quiver with decidable equality on its vertices and arrows, we construct an instance of decidable equality for `Quiver.Path`. We proceed through a recursion on the length of the path utilizing an intermediate subtype of uniformly bounded paths `Quiver.Path.BoundedPath`. This was motivated by doing computations on small quivers with Lean. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 69/0 Mathlib/Combinatorics/Quiver/Path.lean 1 1 ['github-actions'] nobody
0-22514
6 hours ago
0-22603
6 hours ago
0-0
0 seconds
25586 JovanGerb
author:JovanGerb
chore(Order): use new ge/gt naming convention - Part 5 This PR renames, moves around, and deprecates theorems about `PartialOrder`s The main changes are in `Mathlib.Order.Defs.PartialOrder` and `Mathlib.Order.Basic`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 132/121 Mathlib/Algebra/ContinuedFractions/Computation/Approximations.lean,Mathlib/Algebra/Exact.lean,Mathlib/Algebra/Order/AbsoluteValue/Basic.lean,Mathlib/Algebra/Order/BigOperators/Ring/Finset.lean,Mathlib/Algebra/Order/Group/PosPart.lean,Mathlib/Algebra/Order/Group/Unbundled/Abs.lean,Mathlib/Algebra/Order/Monoid/Canonical/Defs.lean,Mathlib/Algebra/Order/Monoid/Unbundled/Basic.lean,Mathlib/Algebra/Order/Ring/Unbundled/Basic.lean,Mathlib/Algebra/Quaternion.lean,Mathlib/Analysis/Analytic/Basic.lean,Mathlib/Analysis/Calculus/Darboux.lean,Mathlib/Analysis/Convex/Gauge.lean,Mathlib/Analysis/Convex/Jensen.lean,Mathlib/Analysis/Convex/Segment.lean,Mathlib/Analysis/InnerProductSpace/Basic.lean,Mathlib/Analysis/InnerProductSpace/LinearMap.lean,Mathlib/Analysis/MeanInequalities.lean,Mathlib/Analysis/Normed/Group/Basic.lean,Mathlib/Analysis/Normed/Group/Continuity.lean,Mathlib/Analysis/Normed/Group/Quotient.lean,Mathlib/Analysis/Normed/Unbundled/RingSeminorm.lean,Mathlib/Analysis/Normed/Unbundled/SeminormFromBounded.lean,Mathlib/Analysis/NormedSpace/Multilinear/Basic.lean,Mathlib/Analysis/NormedSpace/OperatorNorm/Bilinear.lean,Mathlib/Analysis/SpecialFunctions/BinaryEntropy.lean,Mathlib/Analysis/SpecialFunctions/ContinuousFunctionalCalculus/Rpow/IntegralRepresentation.lean,Mathlib/Analysis/SpecialFunctions/Pow/Real.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Inverse.lean,Mathlib/Analysis/SpecificLimits/Normed.lean,Mathlib/Combinatorics/Additive/CauchyDavenport.lean,Mathlib/Combinatorics/Additive/Energy.lean,Mathlib/Combinatorics/Configuration.lean,Mathlib/Combinatorics/SetFamily/FourFunctions.lean,Mathlib/Combinatorics/SimpleGraph/Extremal/Basic.lean,Mathlib/Data/EReal/Operations.lean,Mathlib/Data/Finset/Card.lean,Mathlib/Data/NNReal/Defs.lean,Mathlib/Data/Nat/Find.lean,Mathlib/Data/Set/Sups.lean,Mathlib/FieldTheory/Normal/Closure.lean,Mathlib/Geometry/Euclidean/Angle/Unoriented/Basic.lean,Mathlib/GroupTheory/SpecificGroups/Alternating.lean,Mathlib/LinearAlgebra/Dimension/DivisionRing.lean,Mathlib/LinearAlgebra/FreeModule/PID.lean,Mathlib/LinearAlgebra/Ray.lean,Mathlib/MeasureTheory/Measure/MeasureSpace.lean,Mathlib/NumberTheory/NumberField/CanonicalEmbedding/ConvexBody.lean,Mathlib/NumberTheory/SumFourSquares.lean,Mathlib/Order/Basic.lean,Mathlib/Order/BoundedOrder/Basic.lean,Mathlib/Order/Cover.lean,Mathlib/Order/Defs/PartialOrder.lean,Mathlib/Order/Fin/Basic.lean,Mathlib/Order/Interval/Set/Basic.lean,Mathlib/Order/UpperLower/Closure.lean,Mathlib/RingTheory/ChainOfDivisors.lean,Mathlib/RingTheory/Filtration.lean,Mathlib/RingTheory/Regular/IsSMulRegular.lean,Mathlib/SetTheory/Ordinal/Arithmetic.lean,Mathlib/SetTheory/Ordinal/Family.lean,Mathlib/Topology/Compactness/DeltaGeneratedSpace.lean,Mathlib/Topology/Instances/ENNReal/Lemmas.lean,Mathlib/Topology/Instances/ENat.lean,Mathlib/Topology/MetricSpace/HausdorffDistance.lean,Mathlib/Topology/MetricSpace/Pseudo/Defs.lean,Mathlib/Topology/Neighborhoods.lean,Mathlib/Topology/NhdsSet.lean,Mathlib/Topology/Order.lean 69 3 ['JovanGerb', 'github-actions'] bryangingechen
assignee:bryangingechen
0-22471
6 hours ago
1-29963
1 day ago
1-29947
1 day
25620 paulorauber
author:paulorauber
feat(Probability): sum of sub-Gaussian random variables is sub-Gaussian This shows that the sum of two sub-Gaussian random variables is sub-Gaussian. A previous lemma (`add_of_indepFun`) shows that the sum of two _independent_ sub-Gaussian random variables is sub-Gaussian. --- - The proof of `integrable_exp_mul` is the same as in `add_of_indepFun`, but creating an additional lemma seems excessive. - The positivity requirements (`hcX` and `hcY`) can be eliminated once there is a proof that a 0-subGaussian random variable is zero almost surely. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-measure-probability awaiting-author 31/0 Mathlib/Probability/Moments/SubGaussian.lean 1 5 ['github-actions', 'paulorauber', 'sgouezel'] nobody
0-20628
5 hours ago
0-26865
7 hours ago
0-5071
1 hour
25574 D-Thomine
author:D-Thomine
feat(Cardinal/Finite): ENat powers and cardinality We define the powers of an extended natural number by another extended natural numbers in a new file `Data.Enat.Pow`. We extend `Nat.card_fun` to arbitrary types in `SetTheory.Cardinal.Finite`. - We add a few useful instances (`Pi.nonemptyUnique`, `NoZeroDivisors ℕ∞`, `Subsingleton ℕ∞ˣ`). The latter is in an odd place (`Data.Enat.Pow`), but I did not find a file with the right imports, and did not want to blow up imports in, say, `Data.Enat.Basic`. - This PR has significant overlap with PR #16810 by @urkud . Most of it is convergent evolution (even the names), but I lifted and tweaked the `Pow` instance from there. Overall, I wouldn't mind if we first merged Yuri's PR; it would be better for documenting code contribution, but make for a more complicated process. Another solution would be to add Yuri as an author/copyright holder to `Data.Enat.Pow` if he agrees. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-set-theory t-data 176/1 Mathlib.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/Data/ENat/Pow.lean,Mathlib/Logic/Unique.lean,Mathlib/SetTheory/Cardinal/Finite.lean 5 2 ['github-actions', 'sgouezel'] nobody
0-19715
5 hours ago
1-77362
1 day ago
1-81284
1 day
25527 xroblot
author:xroblot
feat(Data/ZMod): add some simps lemma Add simps lemma to relate the maps constructed here with `Int.castRingHom (ZMod n)` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data t-algebra
label:t-algebra$
20/0 Mathlib/Data/ZMod/QuotientRing.lean 1 3 ['github-actions', 'riccardobrasca', 'xroblot'] nobody
0-19544
5 hours ago
3-40943
3 days ago
3-41033
3 days
24977 YaelDillies
author:YaelDillies
feat(WithZero): `exp : ℤ → ℤₘ₀`, `log : ℤₘ₀ → ℤ` In valuation theory, valuations have codomain `{0} ∪ {e ^ n | n : ℤ}`, which we can formalise as `ℤₘ₀ := WithZero (Multiplicative ℤ)`. It is important to be able to talk about the maps `n ↦ e ^ n` and `e ^ n ↦ n`. We define these as `exp : ℤ → ℤₘ₀` and `log : ℤₘ₀ → ℤ` with junk value `log 0 = 0`. Junkless versions are defined as `expEquiv : ℤ ≃ ℤₘ₀ˣ` and `logEquiv : ℤₘ₀ˣ ≃ ℤ`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
156/36 Mathlib/Algebra/Group/Defs.lean,Mathlib/Algebra/Group/Int/Defs.lean,Mathlib/Algebra/GroupWithZero/Int.lean,Mathlib/Algebra/GroupWithZero/WithZero.lean,Mathlib/Algebra/Order/GroupWithZero/Canonical.lean,Mathlib/Algebra/Order/Ring/IsNonarchimedean.lean,Mathlib/Algebra/Tropical/Basic.lean,Mathlib/RingTheory/Valuation/Discrete/Basic.lean 8 15 ['YaelDillies', 'eric-wieser', 'faenuccio', 'github-actions', 'leanprover-community-bot-assistant', 'pechersky', 'smmercuri'] nobody
0-19141
5 hours ago
0-19162
5 hours ago
22-69464
22 days
25619 xroblot
author:xroblot
feat(NumberField/CMField): A totally complex abelian extension of ℚ is CM --- - [ ] depends on: #23858 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR 165/6 Mathlib/Algebra/Field/Subfield/Basic.lean,Mathlib/FieldTheory/Galois/Basic.lean,Mathlib/FieldTheory/IntermediateField/Adjoin/Basic.lean,Mathlib/FieldTheory/IntermediateField/Basic.lean,Mathlib/LinearAlgebra/Dimension/Finrank.lean,Mathlib/NumberTheory/NumberField/CMField.lean,Mathlib/NumberTheory/NumberField/InfinitePlace/Embeddings.lean 7 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
0-19121
5 hours ago
0-35075
9 hours ago
0-118
1 minute
24796 erdOne
author:erdOne
feat(AlgebraicGeometry): locally directed gluing --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebraic-geometry 480/159 Mathlib.lean,Mathlib/AlgebraicGeometry/Cover/Sigma.lean,Mathlib/AlgebraicGeometry/Gluing.lean,Mathlib/AlgebraicGeometry/IdealSheaf/Subscheme.lean,Mathlib/AlgebraicGeometry/Limits.lean,Mathlib/AlgebraicGeometry/Morphisms/Basic.lean,Mathlib/AlgebraicGeometry/OpenImmersion.lean,Mathlib/AlgebraicGeometry/Restrict.lean,Mathlib/AlgebraicGeometry/Scheme.lean,Mathlib/CategoryTheory/LocallyDirected.lean 10 11 ['chrisflav', 'erdOne', 'github-actions'] nobody
0-19044
5 hours ago
0-19044
5 hours ago
10-9339
10 days
25613 erdOne
author:erdOne
chore(RingTheory/DedekindDomain): missing instances --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
107/3 Mathlib/Algebra/Algebra/Operations.lean,Mathlib/Algebra/Order/GroupWithZero/Unbundled/OrderIso.lean,Mathlib/RingTheory/DedekindDomain/Ideal.lean,Mathlib/RingTheory/FractionalIdeal/Basic.lean 4 1 ['github-actions'] nobody
0-18990
5 hours ago
0-61631
17 hours ago
0-61686
17 hours
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 large-import 726/652 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/Pi/Lemmas.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/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/Lean/Meta/RefinedDiscrTree/Pi.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,scripts/noshake.json 58 11 ['YaelDillies', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
0-18836
5 hours ago
0-18860
5 hours ago
14-16551
14 days
25002 YaelDillies
author:YaelDillies
chore(Finsupp): move order properties under `Order` --- - [ ] depends on: #24998 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) file-removed large-import blocked-by-other-PR 1067/968 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/Pi/Lemmas.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/Data/Finsupp/Basic.lean,Mathlib/Data/Finsupp/Defs.lean,Mathlib/Data/Finsupp/Ext.lean,Mathlib/Data/Finsupp/Order.lean,Mathlib/Data/Finsupp/SMulWithZero.lean,Mathlib/Data/Finsupp/Single.lean,Mathlib/Data/Int/CharZero.lean,Mathlib/Data/Set/Pointwise/Support.lean,Mathlib/GroupTheory/FreeGroup/Basic.lean,Mathlib/Lean/Meta/RefinedDiscrTree/Pi.lean,Mathlib/MeasureTheory/MeasurableSpace/Basic.lean,Mathlib/Order/Filter/Basic.lean,Mathlib/Order/Filter/EventuallyConst.lean,Mathlib/Order/Interval/Set/Pi.lean,Mathlib/Order/Preorder/Finsupp.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,scripts/noshake.json 62 7 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
0-18812
5 hours ago
0-18831
5 hours ago
0-875
14 minutes
25365 YaelDillies
author:YaelDillies
feat: `CommAlgCat` is cocartesian-monoidal Construct the cocartesian-monoidal category structure on `CommAlgCat R` explicitly from the tensor product. From Toric Co-authored-by: Andrew Yang Co-authored-by: Michał Mrugała Co-authored-by: Christian Merten --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) toric t-algebra
label:t-algebra$
142/5 Mathlib.lean,Mathlib/Algebra/Category/CommAlgCat/Basic.lean,Mathlib/Algebra/Category/CommAlgCat/Monoidal.lean 3 8 ['YaelDillies', 'erdOne', 'github-actions'] nobody
0-18718
5 hours ago
7-26981
7 days ago
7-28134
7 days
25584 YaelDillies
author:YaelDillies
chore(Algebra/Order/Module/Defs): don't import fields Instead move the few `Field` lemmas to a new file `Algebra.Order.Module.Field` (https://github.com/leanprover-community/mathlib3/pull/9077 for the copyright) and the `positivity` extension to `Tactic.Positivity.Basic`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 184/153 Archive/Wiedijk100Theorems/InverseTriangleSum.lean,Mathlib.lean,Mathlib/Algebra/GeomSum.lean,Mathlib/Algebra/MvPolynomial/Degrees.lean,Mathlib/Algebra/MvPolynomial/SchwartzZippel.lean,Mathlib/Algebra/Order/AbsoluteValue/Basic.lean,Mathlib/Algebra/Order/BigOperators/Expect.lean,Mathlib/Algebra/Order/CauSeq/Basic.lean,Mathlib/Algebra/Order/CauSeq/BigOperators.lean,Mathlib/Algebra/Order/Floor/Div.lean,Mathlib/Algebra/Order/Hom/Basic.lean,Mathlib/Algebra/Order/Module/Algebra.lean,Mathlib/Algebra/Order/Module/Defs.lean,Mathlib/Algebra/Order/Module/Field.lean,Mathlib/Algebra/Order/Module/OrderedSMul.lean,Mathlib/Algebra/Order/Module/Pointwise.lean,Mathlib/Algebra/Order/Monovary.lean,Mathlib/Algebra/Order/Rearrangement.lean,Mathlib/Combinatorics/Additive/CovBySMul.lean,Mathlib/Data/DFinsupp/Order.lean,Mathlib/Data/Finsupp/Lex.lean,Mathlib/Data/Finsupp/Order.lean,Mathlib/Data/Nat/Factorial/BigOperators.lean,Mathlib/Data/Nat/Factorization/Defs.lean,Mathlib/Data/Nat/Factorization/Induction.lean,Mathlib/Data/Nat/Factorization/Root.lean,Mathlib/Data/Nat/Multiplicity.lean,Mathlib/Data/Nat/Squarefree.lean,Mathlib/Data/Nat/Totient.lean,Mathlib/NumberTheory/FLT/Polynomial.lean,Mathlib/NumberTheory/FactorisationProperties.lean,Mathlib/NumberTheory/FermatPsp.lean,Mathlib/NumberTheory/Padics/PadicNorm.lean,Mathlib/Tactic/Positivity/Basic.lean,scripts/noshake.json 35 3 ['YaelDillies', 'github-actions', 'grunweg'] nobody
0-18484
5 hours ago
0-18492
5 hours ago
0-64021
17 hours
25496 faenuccio
author:faenuccio
feat(Algebra/GroupWithZero/Range): the range of a MonoidHom whose codomain is a GroupWithZero as a GroupWithZero when We define an instance of `GroupWithZero` on the subgroup generated by the range of a MonoidHom taking values in a `GroupWithZero` (by adding a zero to it). Co-authored-by: @AntoineChambert-Loir --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra WIP
label:t-algebra$
265/0 Mathlib/Algebra/GroupWithZero/Range.lean 1 1 ['github-actions'] nobody
0-18462
5 hours ago
2-75464
2 days ago
0-4
4 seconds
24454 robin-carlier
author:robin-carlier
feat(Tactic/CategoryTheory): the `rotate_isos` tactic We define a `rotate_isos` tactic for category theory in mathlib. At its core, the tactic transform terms of type `α(1) ≫ ⋯ ≫ α(k) = β(1) ≫ ⋯ ≫ β(l)` where `α` and `β` are families of morphisms in whith the first `i` morphisms of the left-hand side and the last `j` morphisms of the right-hand side are isomorhisms, into terms of type `α(k-i) ≫ ⋯ ≫ α(k) ≫ inv β(l) ≫ ⋯ ≫ β(l-j+1) = inv α(j) ≫ ⋯ ≫ inv α(1) ≫⋯ ≫ β(l-j)`. The construction of the inverses of expression are caried at the `Expr` levels are built out of the expressions of the morphisms, for instance, for this tactic, the inverse of `F.map (G.map (H.map f.hom)))` will directly be `F.map (G.map (H.map f.inv)))` (which would have to be re-simplified), rather than an `inv` term form an `IsIso` instance. The tactic can be applied at a local hypothesis or at the main goal, or can be used through a `rotate_isos%` term elaborator if e.g one wants to add such a "rotated" form to a `simp` or `rw` call. We also support removing morphisms "from the right" of the lhs, rather than from the right. --- The motivations behind this tactic are the following : - This tactic can "autogenerate" lemmas and terms generalizing lemmas such as [CategoryTheory.Iso.hom_inv_id_app_app_app](https://leanprover-community.github.io/mathlib4_docs/Mathlib/CategoryTheory/NatIso.html#CategoryTheory.Iso.hom_inv_id_app_app_app). This can also generate lemmas `F.map (G.map f.hom) ≫F.map (G.map f.inv) = 𝟙 _`, and can be used to unlock a `simp` call that blocks at an expression of the form `F.map (G.map f.hom) ≫F.map (G.map f.inv) `. - Currently, cancelling morphisms "from the right" in an expression in category theory is a bit of a pain. You have to first reassociate the expression, perform multiple calls to `Iso.inv_comp_eq`, reassociate, etc. This at least automates this process in a fairly straightforward way. - There are expressions in category theory that have no "right forms", e.g the pentagon axiom for monoidal categories, which has many variations in the way one can read the diagram of isomorphisms that represents it. Elaborators such as `rotate_iso%` easily generates all possible forms of such identities from one single form, and avoids having to state multiple forms of the same equality as individual lemmas. - I have been playing with medium-sized diagrams of isomorphisms recently (think for example vertical/horizontal compositions of `CatCommSq`, whiskering a corner of such diagrams, etc.), and it made me wish a lot of time that such easy way to transforms equalities to equivalent forms were available. - [ ] depends on: #24506 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory t-meta awaiting-author blocked-by-other-PR WIP 871/0 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/CategoryTheory/RotateIsos/Cancelable.lean,Mathlib/Tactic/CategoryTheory/RotateIsos/Core.lean,Mathlib/Tactic/CategoryTheory/RotateIsos/Lemmas.lean,MathlibTest/CategoryTheory/RotateIsos.lean,scripts/noshake.json 7 13 ['callesonne', 'github-actions', 'mathlib4-dependent-issues-bot', 'robin-carlier'] nobody
0-18267
5 hours ago
0-20726
5 hours ago
0-495
8 minutes
24845 kebekus
author:kebekus
feat: integrability of log ‖meromorphic‖ For real-meromorphic functions `f`, establish interval integrability of `log ‖f ·‖`. In particular, show that `log ∘ sin` is interval integrable. For complex-meromorphic functions `f`, establish circle integrability of `log ‖f ·‖`. At the suggestion of @sgouezel, split the file [Mathlib/Analysis/SpecialFunctions/Integrals.lean](https://github.com/leanprover-community/mathlib4/pull/24845/files#diff-866dd3a7c4603a1a9d9361ee9e58ea2a97ab83d2037e34d5a8ac23862f421c65). The file establishes values of special interval integrals. As a prerequisite, it establishes interval integrability of numerous functions. Interval integrability of `log ‖f ·‖`, which is established in the current PR, naturally fits in there. Adding the material to [Mathlib/Analysis/SpecialFunctions/Integrals.lean](https://github.com/leanprover-community/mathlib4/pull/24845/files#diff-866dd3a7c4603a1a9d9361ee9e58ea2a97ab83d2037e34d5a8ac23862f421c65) did however not seem advisable: - The line of argumentation is different from what is used already, leading to massive new imports and cross-dependencies. - The current file mixes two lines of results of independent interest that have only a clear one-way dependency (integral computation uses integrability) - The file was very long already. As a clean solution, move the material on integrability to a new directory, `Mathlib/Analysis/SpecialFunctions/Integrability`, which contains a file with the original material and another one with the new material. That way, the results on integrability are all in one place and cross-imports are avoided. 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. Integrability of `log ∘ sin` might be useful in future discussions of polylogarithms. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-measure-probability t-analysis awaiting-author 603/242 Mathlib.lean,Mathlib/Analysis/SpecialFunctions/ExpDeriv.lean,Mathlib/Analysis/SpecialFunctions/Integrability/Basic.lean,Mathlib/Analysis/SpecialFunctions/Integrability/LogMeromorphic.lean,Mathlib/Analysis/SpecialFunctions/Integrals.lean,Mathlib/Analysis/SpecialFunctions/JapaneseBracket.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Deriv.lean,Mathlib/MeasureTheory/Integral/CircleIntegral.lean,Mathlib/MeasureTheory/Integral/IntervalIntegral/Basic.lean 9 39 ['Ruben-VandeVelde', 'github-actions', 'grunweg', 'kebekus', 'leanprover-community-bot-assistant', 'sgouezel'] nobody
0-18242
5 hours ago
0-18242
5 hours ago
19-28075
19 days
24823 eric-wieser
author:eric-wieser
refactor: add `hom` lemmas for the `MonoidalCategory` structure on `ModuleCat` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
148/164 Mathlib/Algebra/Category/FGModuleCat/Basic.lean,Mathlib/Algebra/Category/ModuleCat/Adjunctions.lean,Mathlib/Algebra/Category/ModuleCat/Monoidal/Basic.lean,Mathlib/Algebra/Category/ModuleCat/Monoidal/Closed.lean,Mathlib/Algebra/Category/ModuleCat/Monoidal/Symmetric.lean,Mathlib/Algebra/Category/ModuleCat/Presheaf/Free.lean,Mathlib/Algebra/Category/ModuleCat/Presheaf/Generator.lean,Mathlib/Algebra/Category/ModuleCat/Presheaf/Monoidal.lean,Mathlib/CategoryTheory/Monoidal/Internal/Module.lean,Mathlib/RepresentationTheory/Coinvariants.lean,Mathlib/RepresentationTheory/Rep.lean 11 20 ['101damnations', 'YaelDillies', 'eric-wieser', 'github-actions', 'joelriou', 'kbuzzard', 'leanprover-community-bot-assistant'] 101damnations
assignee:101damnations
0-17659
4 hours ago
0-17678
4 hours ago
18-13725
18 days
25309 101damnations
author:101damnations
feat(RepresentationTheory): `Ind` and `Coind` isomorphism for a finite index subgroup Given a commutative ring `k`, a finite index subgroup `S ≤ G`, and a `k`-linear `S`-representation `A`, this PR defines an isomorphism $Ind_S^G(A) ≅ Coind_S^G(A).$ Given `g : G` and `a : A`, the forward map sends `⟦g ⊗ₜ[k] a⟧` to the function `G → A`supported at `sg` by `ρ(s)(a)` for `s : S` and which is 0 elsewhere. Meanwhile, the inverse sends `f : G → A` to `∑ᵢ ⟦gᵢ ⊗ₜ[k] f(gᵢ)⟧` for `1 ≤ i ≤ n`, where `g₁, ..., gₙ` is a set of right coset representatives of `S`. --- - [x] depends on: #21732 - [x] depends on: #21733 - [x] depends on: #21735 - [x] depends on: #25307 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
259/0 Mathlib.lean,Mathlib/RepresentationTheory/Shapiro.lean 2 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
0-17408
4 hours ago
0-17408
4 hours ago
0-17401
4 hours
25611 erdOne
author:erdOne
chore(RingTheory): add `Algebra (FractionRing R) (FractionRing S)` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
113/108 Mathlib.lean,Mathlib/Algebra/Algebra/NonZeroDivisors.lean,Mathlib/NumberTheory/RamificationInertia/Galois.lean,Mathlib/RingTheory/DedekindDomain/Different.lean,Mathlib/RingTheory/DedekindDomain/IntegralClosure.lean,Mathlib/RingTheory/Ideal/Norm/RelNorm.lean,Mathlib/RingTheory/IntegralClosure/IntegralRestrict.lean,Mathlib/RingTheory/Localization/FractionRingAlgebra.lean,Mathlib/RingTheory/Localization/Integral.lean 9 6 ['erdOne', 'eric-wieser', 'github-actions'] nobody
0-16100
4 hours ago
0-47505
13 hours ago
0-62245
17 hours
25591 erdOne
author:erdOne
feat(RingTheory/DedekindDomain): residue field extension not separable implies divides different --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-algebra
label:t-algebra$
159/7 Mathlib/FieldTheory/PurelyInseparable/Basic.lean,Mathlib/RingTheory/DedekindDomain/Different.lean,Mathlib/RingTheory/Trace/Basic.lean 3 1 ['github-actions'] nobody
0-15923
4 hours ago
1-20822
1 day ago
1-20904
1 day
25622 eric-wieser
author:eric-wieser
refactor: overhaul instances on LocalizedModule This: * Generalizes the `SMul`, `Module`, and `Algebra` instances via appropriate compatibility conditions * Generalizes the `Mul` instance to the non-unital setting * Fixes instances diamonds for the `Nat`- and `Int`-actions --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
167/111 Mathlib/Algebra/Module/LocalizedModule/Basic.lean 1 3 ['erdOne', 'eric-wieser', 'github-actions'] nobody
0-15780
4 hours ago
0-16397
4 hours ago
0-23650
6 hours
25606 adomani
author:adomani
fix(CI): make autolabel run on `pull_request_target` Mentioned by Bryan [here](https://github.com/leanprover-community/mathlib4/pull/25599#issuecomment-2954240919). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) CI awaiting-author 10/2 .github/workflows/add_label_from_diff.yaml 1 3 ['bryangingechen', 'github-actions', 'mattrobball'] nobody
0-15576
4 hours ago
0-81570
22 hours ago
0-3768
1 hour
25417 Timeroot
author:Timeroot
feat(Analysis/InnerProductSpace): exchange range + ker ``` theorem range_le_range_iff_ker_le_ker {U : E →ₗ[𝕜] E} (hT : T.IsSymmetric) (hU : U.IsSymmetric) : range T ≤ range U ↔ ker U ≤ ker T := by ``` and the forward direction holds in the infinite dimensional case too. Upstreamed from [quantumInfo](https://github.com/Timeroot/Lean-QuantumInfo) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis awaiting-author 68/13 Mathlib/Analysis/Convex/Basic.lean,Mathlib/Analysis/InnerProductSpace/Adjoint.lean,Mathlib/Analysis/InnerProductSpace/Orthogonal.lean,Mathlib/Analysis/InnerProductSpace/Projection.lean,Mathlib/Analysis/InnerProductSpace/Symmetric.lean 5 18 ['Timeroot', 'github-actions', 'j-loreaux'] nobody
0-15010
4 hours ago
0-15010
4 hours ago
0-52027
14 hours
25310 101damnations
author:101damnations
refactor(RepresentationTheory/GroupCohomology): refactor low degree group cohomology --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra WIP
label:t-algebra$
617/404 Mathlib/Algebra/Homology/ShortComplex/ModuleCat.lean,Mathlib/RepresentationTheory/GroupCohomology/Basic.lean,Mathlib/RepresentationTheory/GroupCohomology/Functoriality.lean,Mathlib/RepresentationTheory/GroupCohomology/Hilbert90.lean,Mathlib/RepresentationTheory/GroupCohomology/LowDegree.lean,Mathlib/RepresentationTheory/Rep.lean 6 2 ['github-actions', 'leanprover-community-bot-assistant'] nobody
0-14858
4 hours ago
0-17959
4 hours ago
0-12
12 seconds
25523 kebekus
author:kebekus
feat: compute trailing coefficients of factorized rational functions Compute the trailing coefficient of factorized rational functions. Apply this to compute the trailing coefficient of arbitrary meromorphic functions, presented as a product of a factorized rational and an analytic function. 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. It is one of the ingredients in the proof of Jensen's Formula in complex analysis. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis 177/3 Mathlib/Analysis/Meromorphic/FactorizedRational.lean,Mathlib/Analysis/Meromorphic/TrailingCoefficient.lean 2 2 ['github-actions', 'sgouezel'] nobody
0-11170
3 hours ago
3-46984
3 days ago
3-47054
3 days
25625 vlad902
author:vlad902
feat(data): List.Chain' helper lemmas Add two helpers lemmas to go from a positive/negative List.Chain' hypothesis to a concrete goal about two consecutive elements of the list. t-data 22/0 Mathlib/Data/List/Chain.lean 1 1 ['github-actions'] nobody
0-10531
2 hours ago
0-10706
2 hours ago
0-10690
2 hours
25144 wwylele
author:wwylele
feat(Algebra/Order): add Archimedean class This is the first of PRs for Hahn embedding theorem #25140 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
442/0 Mathlib.lean,Mathlib/Algebra/Order/Archimedean/Class.lean,Mathlib/Algebra/Order/Group/Unbundled/Abs.lean 3 49 ['YaelDillies', 'eric-wieser', 'github-actions', 'wwylele'] nobody
0-10157
2 hours ago
0-78434
21 hours ago
16-42508
16 days
25609 Multramate
author:Multramate
feat(Algebra/Group/Units/Hom): add map lemmas --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-algebra easy
label:t-algebra$
21/10 Mathlib/Algebra/Group/Units/Defs.lean,Mathlib/Algebra/Group/Units/Hom.lean 2 15 ['Multramate', 'erdOne', 'github-actions'] nobody
0-9828
2 hours ago
0-9828
2 hours ago
0-9813
2 hours
25010 emilyriehl
author:emilyriehl
the homotopy category functor preserves products This is work in progress with several sorries. Co-authored-by: Dominic Verity and Thomas Murrills --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) infinity-cosmos large-import t-category-theory WIP 352/4 Mathlib/AlgebraicTopology/SimplexCategory/Basic.lean,Mathlib/AlgebraicTopology/SimplicialSet/HoFunctorPreservesBinaryProducts.lean,Mathlib/AlgebraicTopology/SimplicialSet/Monoidal.lean,Mathlib/CategoryTheory/ComposableArrows.lean,Mathlib/CategoryTheory/PUnit.lean 5 2 ['github-actions'] nobody
0-8426
2 hours ago
6-78765
6 days ago
0-45
45 seconds
24575 pfaffelh
author:pfaffelh
feat: introduce Gram matrices A Gram matrix has entry `⟪v i, v j⟫` at `i j : n`, where `v : n → α` is an `InnerProductSpace 𝕜 α`. Give this notion and show that Gram matrices are positive semi-definite. This will be used later in order to show that the covariance matrix for Brownian Motion is positive semi-definite. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-measure-probability awaiting-author 233/0 Mathlib.lean,Mathlib/Analysis/InnerProductSpace/GramMatrix.lean,Mathlib/MeasureTheory/Function/L2Space.lean,Mathlib/Probability/Process/BrownianMotion.lean 4 98 ['eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'pfaffelh', 'sgouezel'] nobody
0-6958
1 hour ago
0-39923
11 hours ago
20-66528
20 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$
477/61 Mathlib/Algebra/Algebra/Pi.lean,Mathlib/Algebra/Ring/Equiv.lean,Mathlib/LinearAlgebra/DFinsupp.lean,Mathlib/Order/CompleteSublattice.lean,Mathlib/RingTheory/SimpleModule/Basic.lean,Mathlib/RingTheory/SimpleModule/IsAlgClosed.lean,Mathlib/RingTheory/SimpleModule/Isotypic.lean,Mathlib/RingTheory/SimpleModule/WedderburnArtin.lean 8 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
0-6831
1 hour ago
0-6877
1 hour ago
22-85358
22 days
24983 alreadydone
author:alreadydone
fix(Topology/Covering): switch to standard definition As discussed in [#mathlib4 > edge cases not covered by `IsCoveringMap` @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/edge.20cases.20not.20covered.20by.20.60IsCoveringMap.60/near/518413081), the previous definition doesn't include examples like the inclusion of a one-point space into a two-point discrete space. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology 168/54 Mathlib/Topology/Covering.lean,Mathlib/Topology/FiberBundle/Trivialization.lean,Mathlib/Topology/Homotopy/Lifting.lean 3 6 ['alreadydone', 'github-actions', 'leanprover-community-bot-assistant', 'tb65536'] nobody
0-6803
1 hour ago
0-6865
1 hour ago
20-50511
20 days
25626 robin-carlier
author:robin-carlier
feat(CategoryTheory/Monoidal/Opposites): monoid objects internal to the monoidal opposite We construct an equivalence between monoid objects internal to a monoidal category `C`, and monoid objects internal to its monoidal opposite `Cᴹᵒᵖ`. This is done by adding `Mon_Class` and `IsMon_Hom` instance to the relevant objects, as well as by recording an explicit equivalence of categories `Mon_ C ≌ Mon_ Cᴹᵒᵖ`. --- - [ ] depends on: #25549 I made this depend on #25549 rather than making it work with the current def only to have it refactored when #25549 is merged. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory blocked-by-other-PR 321/173 Mathlib.lean,Mathlib/Algebra/Category/CoalgCat/ComonEquivalence.lean,Mathlib/CategoryTheory/Monad/EquivMon.lean,Mathlib/CategoryTheory/Monoidal/Bimon_.lean,Mathlib/CategoryTheory/Monoidal/Cartesian/Comon_.lean,Mathlib/CategoryTheory/Monoidal/Cartesian/Mon_.lean,Mathlib/CategoryTheory/Monoidal/CommGrp_.lean,Mathlib/CategoryTheory/Monoidal/CommMon_.lean,Mathlib/CategoryTheory/Monoidal/Comon_.lean,Mathlib/CategoryTheory/Monoidal/Grp_.lean,Mathlib/CategoryTheory/Monoidal/Internal/FunctorCategory.lean,Mathlib/CategoryTheory/Monoidal/Internal/Limits.lean,Mathlib/CategoryTheory/Monoidal/Internal/Module.lean,Mathlib/CategoryTheory/Monoidal/Internal/Types/Basic.lean,Mathlib/CategoryTheory/Monoidal/Mod_.lean,Mathlib/CategoryTheory/Monoidal/Mon_.lean,Mathlib/CategoryTheory/Monoidal/Opposite/Mon_.lean,Mathlib/CategoryTheory/Preadditive/CommGrp_.lean 18 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
0-6370
1 hour ago
0-6370
1 hour ago
0-1460
24 minutes
24778 YaelDillies
author:YaelDillies
feat: `CommGrp`-valued Yoneda embedding From Toric Co-authored-by: Andrew Yang --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) toric large-import t-category-theory awaiting-author 65/6 Mathlib/Algebra/Category/Grp/Basic.lean,Mathlib/Algebra/Category/Grp/ForgetCorepresentable.lean,Mathlib/Algebra/Category/MonCat/Basic.lean,Mathlib/Algebra/Category/MonCat/ForgetCorepresentable.lean,Mathlib/CategoryTheory/Preadditive/Yoneda/Basic.lean 5 7 ['TwoFX', 'YaelDillies', 'callesonne', 'github-actions', 'leanprover-community-bot-assistant'] nobody
0-6365
1 hour ago
0-8567
2 hours ago
27-7755
27 days
25491 tannerduve
author:tannerduve
feat(Control/Monad/Freer): define freer monad, prove it lawful, and implement standard effects **Description:** This PR introduces the `Free` monad. This implementation uses the "freer monad" approach as the traditional free monad (eg from [Haskell](https://hackage.haskell.org/package/free-5.2/docs/Control-Monad-Free.html)) is not safely definable in Lean due to termination checking (it's not strictly positive). The main contributions are: * Definition of the `Free` monad as an inductive type which generates a monad given any type constructor `F : Type -> Type`. * Functor and Monad instances for `Free F`, along with proofs of the `LawfulFunctor` and `LawfulMonad` laws. * Canonical instances of `Free` with standard effect signatures: * `FreeState s` for stateful computations, defined via a `StateF s` functor with `get` and `put` operations. * `FreeWriter w` for logging computations, defined via a `WriterF w` functor with a `tell` operation. * `FreeCont r` for continuation-passing computations, using the CPS functor `(α → r) → r`. In this construction, computations are represented as **trees of effects**. Each node (`liftBind`) represents a request to perform an effect, accompanied by a continuation specifying how the computation proceeds after the effect. The leaves (`pure`) represent completed computations with final results. A key insight is that `FreeM F` satisfies the **universal property of free monads**: for any monad `M` and effect handler `f : F → M`, there exists a unique way to interpret `FreeM F` computations in `M` that respects the effect semantics given by `f`. This unique interpreter is `mapM f`, which acts as the canonical **fold** (catamorphism) for free monads. To execute or interpret these computations, we provide two approaches: 1. **Hand-written interpreters** (`FreeState.run`, `FreeWriter.run`, `FreeCont.run`) that directly pattern-match on the tree structure 2. **Canonical interpreters** (`FreeState.fold`, `FreeWriter.fold`, `FreeCont.fold`) derived from the universal property via `mapM` And then prove that these approaches are equivalent **Footer:** 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 696/0 Mathlib.lean,Mathlib/Control/Monad/Free.lean,MathlibTest/freemonad.lean,docs/references.bib 4 79 ['copilot-pull-request-reviewer', 'eric-wieser', 'github-actions', 'plp127', 'quangvdao', 'tannerduve'] nobody
0-5980
1 hour ago
2-82705
2 days ago
4-4789
4 days
25168 wwylele
author:wwylele
feat(RingTheorey/HahnSeries): equip HahnSeries with LinearOrder This is part of #25140. As the future codomain of Hahn embedding theorem, `HahnSeries` needs a linear order. ~~It might be debatable whether the lexicographical order should be *the* order of `HahnSeries`. Aside from usage in Hahn embedding theorem, this order also represents, for example, the asymptotic behavior around `(x : R) = 0`, so it is generally useful.~~ Updated to add `LinearOrder` on `Lex (HahnSeries _ _)` instead --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
180/0 Mathlib.lean,Mathlib/RingTheory/HahnSeries/Addition.lean,Mathlib/RingTheory/HahnSeries/Basic.lean,Mathlib/RingTheory/HahnSeries/Lex.lean 4 10 ['ScottCarnahan', 'eric-wieser', 'github-actions', 'wwylele'] nobody
0-5576
1 hour ago
15-72780
15 days ago
15-72831
15 days
25455 ADedecker
author:ADedecker
feat: refactor and expand lemmas about integration and continuous functional calculus --- - [ ] depends on: #25458 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis blocked-by-other-PR 807/80 Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Integral.lean,Mathlib/MeasureTheory/Function/L1Space/HasFiniteIntegral.lean,Mathlib/MeasureTheory/Function/L1Space/Integrable.lean,Mathlib/MeasureTheory/Integral/IntegrableOn.lean 4 7 ['ADedecker', 'dupuisf', 'github-actions', 'j-loreaux', 'mathlib4-dependent-issues-bot'] nobody
0-4993
1 hour ago
4-81292
4 days ago
0-0
0 seconds
8977 eric-wieser
author:eric-wieser
testing for leanprover/lean4#2940 (`extends flat`) This can be used as a base commit for other branches testing the effect of `extends flat`. This tests leanprover/lean4#2940 Experiments to try: * What happens if we make `class SomeHomClass` flat? (https://github.com/leanprover-community/mathlib4/pull/8978) * What happens if we make `structure SomeHomClass` flat? (#6791, but needs adapting to the keyword) * What happens if we make (some of) the algebraic hierarchy flat? Unfortunately flat `class`es will run up against https://github.com/leanprover/lean4/pull/2905, so the performance change may be difficult to measure in isolation. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP 1/1 lean-toolchain 1 2 ['eric-wieser', 'leanprover-bot'] nobody
546-18780
1 year ago
546-18943
1 year ago
0-0
0 seconds
13158 erdOne
author:erdOne
refactor(RingTheory/OreLocalization/Module): remove `LocalizedModule.mk`. --- - [x] depends on: #13151 - [ ] depends on: #13156 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict blocked-by-other-PR
label:t-algebra$
49/48 Mathlib/RingTheory/OreLocalization/Basic.lean,Mathlib/RingTheory/OreLocalization/Module.lean 2 1 ['leanprover-community-mathlib4-bot'] nobody
335-23447
11 months ago
335-23470
11 months ago
0-0
0 seconds
14720 eric-wieser
author:eric-wieser
refactor: change `CliffordAlgebra.lift` to use quadratic maps This works towards addressing a footnote on [page 152](https://eric-wieser.github.io/thesis/eric-wieser-thesis.pdf#page=164) of my thesis. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict WIP
label:t-algebra$
200/167 Mathlib/LinearAlgebra/CliffordAlgebra/Basic.lean,Mathlib/LinearAlgebra/CliffordAlgebra/Equivs.lean,Mathlib/LinearAlgebra/CliffordAlgebra/Prod.lean,Mathlib/LinearAlgebra/QuadraticForm/Complex.lean,Mathlib/LinearAlgebra/QuadraticForm/Dual.lean,Mathlib/LinearAlgebra/QuadraticForm/Isometry.lean,Mathlib/LinearAlgebra/QuadraticForm/IsometryEquiv.lean,Mathlib/LinearAlgebra/QuadraticForm/Prod.lean,Mathlib/LinearAlgebra/QuadraticForm/QuadraticModuleCat.lean,Mathlib/LinearAlgebra/QuadraticForm/Real.lean,Mathlib/LinearAlgebra/QuadraticForm/TensorProduct/Isometries.lean 11 1 ['github-actions'] nobody
313-42773
10 months ago
327-33768
10 months ago
0-0
0 seconds
14889 yuma-mizuno
author:yuma-mizuno
feat(CategoryTheory/Bicategory/Monad): define monad in bicategory --- - [ ] depends on: #12107 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory merge-conflict blocked-by-other-PR WIP 1566/12 Mathlib.lean,Mathlib/CategoryTheory/Bicategory/Functor/Oplax.lean,Mathlib/CategoryTheory/Bicategory/LocallyDiscrete.lean,Mathlib/CategoryTheory/Bicategory/Monad/Adjunction.lean,Mathlib/CategoryTheory/Bicategory/Monad/Basic.lean,Mathlib/CategoryTheory/Bicategory/Monad/Cat.lean,Mathlib/CategoryTheory/Monad/Basic.lean,Mathlib/Tactic.lean,Mathlib/Tactic/CategoryTheory/Coherence.lean,Mathlib/Tactic/Widget/StringDiagram.lean,scripts/noshake.json,test/StringDiagram.lean,widget/src/penrose/monoidal.dsl,widget/src/penrose/monoidal.sty 14 2 ['github-actions', 'leanprover-community-mathlib4-bot'] nobody
313-42773
10 months ago
325-54011
10 months ago
0-0
0 seconds
14426 adomani
author:adomani
dev: `#min_imps` command --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP 142/0 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/MinImports.lean,test/MinImports.lean 4 2 ['adomani', 'github-actions'] nobody
313-42773
10 months ago
326-39154
10 months ago
0-0
0 seconds
14130 Multramate
author:Multramate
feat(AlgebraicGeometry/EllipticCurve/Scheme): define the affine scheme associated to an elliptic curve This contribution was created as part of the AIM workshop "Formalizing Algebraic Geometry" in June 2024. Co-authored-by: Michael Stoll Co-authored-by: Junyan Xu --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) workshop-AIM-AG-2024 t-algebraic-geometry t-number-theory merge-conflict awaiting-author WIP 557/22 Mathlib/Algebra/DirectSum/Basic.lean,Mathlib/Algebra/DirectSum/Module.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Scheme.lean,Mathlib/RingTheory/GradedAlgebra/Basic.lean,Mathlib/RingTheory/MvPolynomial/Homogeneous.lean,Mathlib/RingTheory/MvPolynomial/WeightedHomogeneous.lean 6 3 ['Multramate', 'github-actions', 'jcommelin'] nobody
313-42772
10 months ago
325-20368
10 months ago
0-0
0 seconds
13847 alreadydone
author:alreadydone
feat(EllipticCurve): the universal elliptic curve + Define the universal Weierstrass curve (`Universal.curve`) over the polynomial ring `ℤ[A₁,A₂,A₃,A₄,A₆]`, and the universal pointed elliptic curve (`Universal.pointedCurve`) over the field of fractions (`Universal.Field`) of the universal ring `ℤ[A₁,A₂,A₃,A₄,A₆,X,Y]/⟨P⟩ = Universal.Poly/⟨P⟩` (`Universal.Ring`, where `P` is the Weierstrass polynomial) with distinguished point `(X,Y)`. + Given a Weierstrass curve `W` over a commutative ring `R`, we define the specialization homomorphism `W.specialize : ℤ[A₁,A₂,A₃,A₄,A₆] →+* R`. If `(x,y)` is a point on the affine plane, we define `W.polyEval x y : Universal.Poly →+* R`, which factors through `W.ringEval x y : Universal.Ring →+* R` if `(x,y)` is on `W`. + Introduce the cusp curve `Y² = X³`, on which lies the rational point `(1,1)`, with the nice property that `ψₙ(1,1) = n`, making it easy to prove nonvanishing of the universal `ψₙ` when `n ≠ 0` by specializing to the cusp curve, which shows that `(X,Y)` is a point of infinite order on the universal pointed elliptic curve. --- - [x] depends on: #13845 - [x] depends on: #12883 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-algebraic-geometry merge-conflict awaiting-author
label:t-algebra$
543/208 Mathlib.lean,Mathlib/Algebra/Polynomial/Bivariate.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Affine.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Group.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Jacobian.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Universal.lean 6 4 ['Multramate', 'alreadydone', 'github-actions', 'leanprover-community-mathlib4-bot'] nobody
313-42772
10 months ago
346-69469
11 months ago
0-0
0 seconds
14036 adomani
author:adomani
Test/decl diff in lean --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict 465/1040 .github/workflows/Lean_decl_diff.yml,.github/workflows/bors.yml,.github/workflows/build.yml,.github/workflows/build.yml.in,.github/workflows/build_fork.yml,.github/workflows/mk_build_yml.sh,scripts/decls_diff_hybrid.sh,scripts/list_decls.lean 8 1 ['github-actions'] nobody
313-42772
10 months ago
351-41063
11 months ago
0-0
0 seconds
14167 alreadydone
author:alreadydone
feat: Group scheme structure on Weierstrass curve --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) workshop-AIM-AG-2024 t-algebraic-geometry merge-conflict WIP 727/41 Mathlib.lean,Mathlib/Algebra/GroupWithZero/NonZeroDivisors.lean,Mathlib/Algebra/Polynomial/Bivariate.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Group.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Scheme.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Universal.lean,Mathlib/Data/Finsupp/Basic.lean,Mathlib/GroupTheory/MonoidLocalization.lean,Mathlib/LinearAlgebra/Basis.lean,Mathlib/LinearAlgebra/FreeModule/Basic.lean,Mathlib/RingTheory/AlgebraTower.lean,Mathlib/RingTheory/MvPolynomial/Basic.lean 12 3 ['Multramate', 'github-actions', 'jcommelin'] nobody
313-42772
10 months ago
326-30383
10 months ago
0-0
0 seconds
13297 urkud
author:urkud
feat(Semicontinuous): add `comp` lemma --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order t-topology merge-conflict awaiting-author 31/13 Mathlib/Topology/Semicontinuous.lean 1 3 ['sgouezel', 'urkud'] nobody
313-42771
10 months ago
325-20502
10 months ago
0-18175
5 hours
13372 adomani
author:adomani
dev: generic replacement --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict 446/0 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter/ReplaceRefine.lean,Mathlib/Tactic/Replacements.lean 4 4 ['adomani', 'github-actions'] nobody
313-42771
10 months ago
355-37680
11 months ago
0-0
0 seconds
13512 adomani
author:adomani
test: count all --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict 85/0 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter.lean,Mathlib/Tactic/Linter/Tally.lean 4 0 [] nobody
313-42771
10 months ago
355-37553
11 months ago
0-0
0 seconds
13057 alreadydone
author:alreadydone
feat(NumberTheory): characterize elliptic divisibility sequences Main results: + Every `normEDS` is an elliptic divisibility sequence (EDS). The key proof is `rel₄_of_anti_oddRec_evenRec`, based on my original argument first published on [MathSE](https://math.stackexchange.com/a/4903422/12932) + Conversely, every EDS is equal to some `normEDS` (assuming that the first two terms are not zero divisors) --- - [ ] depends on: #13155 - [x] depends on: #13153 - [x] depends on: #10843 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-number-theory merge-conflict blocked-by-other-PR
label:t-algebra$
1032/55 Mathlib/Algebra/Ring/NegOnePow.lean,Mathlib/Data/Int/Defs.lean,Mathlib/Data/Int/Parity.lean,Mathlib/GroupTheory/Perm/Sign.lean,Mathlib/NumberTheory/EllipticDivisibilitySequence.lean 5 6 ['Multramate', 'alreadydone', 'kbuzzard', 'leanprover-community-mathlib4-bot'] nobody
313-42770
10 months ago
363-84158
11 months ago
0-34665
9 hours
12933 grunweg
author:grunweg
chore: replace some use of > or ≥ by < or ≤ These were flagged by the linter in #12879: it is easy to simple avoid > or ≥ in hypotheses or `have`s. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author 123/123 Archive/Imo/Imo1960Q1.lean,Archive/Imo/Imo1962Q1.lean,Archive/Imo/Imo1988Q6.lean,Archive/Imo/Imo2005Q3.lean,Archive/Imo/Imo2008Q2.lean,Archive/Imo/Imo2008Q4.lean,Archive/Imo/Imo2011Q5.lean,Archive/Imo/Imo2019Q4.lean,Archive/Wiedijk100Theorems/AreaOfACircle.lean,Archive/Wiedijk100Theorems/BallotProblem.lean,Mathlib/Algebra/DualNumber.lean,Mathlib/Algebra/Order/CauSeq/BigOperators.lean,Mathlib/Algebra/Order/Ring/Defs.lean,Mathlib/Algebra/Polynomial/Basic.lean,Mathlib/Algebra/Polynomial/Degree/Definitions.lean,Mathlib/Algebra/Star/CHSH.lean,Mathlib/Analysis/Analytic/Basic.lean,Mathlib/Analysis/Calculus/UniformLimitsDeriv.lean,Mathlib/Analysis/Complex/Hadamard.lean,Mathlib/Analysis/Complex/UpperHalfPlane/Basic.lean,Mathlib/Analysis/InnerProductSpace/Projection.lean,Mathlib/Analysis/Normed/Group/ControlledClosure.lean,Mathlib/Analysis/SpecialFunctions/Log/Base.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Basic.lean,Mathlib/Combinatorics/SimpleGraph/DegreeSum.lean,Mathlib/Combinatorics/SimpleGraph/LapMatrix.lean,Mathlib/Data/Complex/Basic.lean,Mathlib/Data/FP/Basic.lean,Mathlib/Data/Finset/Basic.lean,Mathlib/Data/Finsupp/Notation.lean,Mathlib/Data/Nat/Dist.lean,Mathlib/Data/Nat/Lattice.lean,Mathlib/Data/Nat/Parity.lean,Mathlib/Data/Ordmap/Ordset.lean,Mathlib/Data/PNat/Basic.lean,Mathlib/Data/UInt.lean,Mathlib/GroupTheory/Coxeter/Length.lean,Mathlib/MeasureTheory/Constructions/Polish.lean,Mathlib/MeasureTheory/Covering/Besicovitch.lean,Mathlib/MeasureTheory/Covering/Vitali.lean,Mathlib/MeasureTheory/Covering/VitaliFamily.lean,Mathlib/MeasureTheory/Integral/Layercake.lean,Mathlib/NumberTheory/LegendreSymbol/JacobiSymbol.lean,Mathlib/NumberTheory/Padics/Hensel.lean,Mathlib/NumberTheory/Padics/PadicNorm.lean,Mathlib/NumberTheory/PellMatiyasevic.lean,Mathlib/NumberTheory/Rayleigh.lean,Mathlib/Probability/Process/Stopping.lean,Mathlib/Tactic/CancelDenoms/Core.lean,Mathlib/Tactic/IntervalCases.lean,Mathlib/Tactic/Linarith/Lemmas.lean,Mathlib/Tactic/Linarith/Oracle/FourierMotzkin.lean,Mathlib/Tactic/NormNum/GCD.lean,Mathlib/Tactic/NormNum/Inv.lean,Mathlib/Tactic/Ring/Basic.lean,Mathlib/Topology/Category/Profinite/Nobeling.lean,Mathlib/Topology/ContinuousFunction/Bounded.lean,Mathlib/Topology/MetricSpace/CauSeqFilter.lean,Mathlib/Topology/Sequences.lean,test/LibrarySearch/basic.lean,test/Use.lean,test/cancel_denoms.lean,test/linarith.lean,test/norm_cast.lean 64 6 ['YaelDillies', 'github-actions', 'grunweg'] nobody
313-42770
10 months ago
326-52361
10 months ago
0-55655
15 hours
12465 rosborn
author:rosborn
style: Change Subtype.val to (↑) --- This is a test to see replacing `Subtype.val` with `(↑)` where appropriate. After performing the rewrite, some of the types subtly changed in a difficult to detect manner. Before the change, `openEmbedding' _` had type `OpenEmbedding Subtype.val` where `Subtype.val` expanded as `@Subtype.val α fun x ↦ x ∈ U : ↥U → α`. After the change, `Subtype.val` expands to `@Subtype.val α fun x ↦ x ∈ ↑U : { x // x ∈ ↑U } → α`. This caused some later proofs to fail due to the different definition. In a similar case, within the proof of `mfderiv_coe_sphere_injective` on line 553 `Subtype.val` expanded as `@Subtype.val E fun x ↦ x ∈ (Submodule.span ℝ {↑(-v)})ᗮ : ↥(Submodule.span ℝ {↑(-v)})ᗮ → E`. After changing to `(↑)`, it expanded to `@Subtype.val E fun x ↦ x ∈ ↑(Submodule.span ℝ {↑(-v)})ᗮ : { x // x ∈ ↑(Submodule.span ℝ {↑(-v)})ᗮ } → E`. One benefit to using `(↑)` was that it lead to a shorter proof as `ContinuousLinearEquiv.coe_coe` could be removed on line 559. In general, this subtle change in types is basically impossible to detect without a tool like leaff. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict 50/50 Mathlib/Analysis/InnerProductSpace/Basic.lean,Mathlib/Analysis/Normed/Group/Hom.lean,Mathlib/CategoryTheory/Generator.lean,Mathlib/CategoryTheory/Limits/Shapes/Types.lean,Mathlib/CategoryTheory/Subobject/Types.lean,Mathlib/Data/Fin/Basic.lean,Mathlib/Data/Set/Function.lean,Mathlib/Data/Set/Image.lean,Mathlib/Data/Setoid/Basic.lean,Mathlib/Geometry/Manifold/ContMDiff/Basic.lean,Mathlib/Geometry/Manifold/Instances/Sphere.lean,Mathlib/Geometry/Manifold/LocalInvariantProperties.lean,Mathlib/GroupTheory/Subsemigroup/Operations.lean,Mathlib/LinearAlgebra/LinearIndependent.lean,Mathlib/Order/Directed.lean,Mathlib/Order/RelIso/Basic.lean,Mathlib/Order/RelIso/Set.lean,Mathlib/RingTheory/Artinian.lean,Mathlib/SetTheory/Cardinal/Cofinality.lean,Mathlib/SetTheory/Game/Basic.lean,Mathlib/SetTheory/Game/PGame.lean,Mathlib/SetTheory/Surreal/Basic.lean,Mathlib/Topology/Bornology/Constructions.lean,Mathlib/Topology/EMetricSpace/Lipschitz.lean,Mathlib/Topology/Germ.lean,Mathlib/Topology/UniformSpace/Basic.lean,Mathlib/Topology/UniformSpace/UniformConvergenceTopology.lean,Mathlib/Topology/UniformSpace/UniformEmbedding.lean 28 1 ['eric-wieser', 'rosborn'] nobody
313-42770
10 months ago
402-18561
1 year ago
0-0
0 seconds
12528 adomani
author:adomani
test: autotranslations Bot --> Top --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict 350/294 Mathlib.lean,Mathlib/Order/WithBot.lean,Mathlib/Tactic.lean,Mathlib/Tactic/MinMax.lean,test/MinMax.lean 5 0 [] nobody
313-42770
10 months ago
383-42912
1 year ago
0-0
0 seconds
12936 mattrobball
author:mattrobball
chore(Quiver.Opposite): make `Quiver.Hom.op/unop` `abbrev`'s These are wrappers around the constructor and projection for `Opposite Quiver.Hom _ _`. The projection itself is reducible and with structure eta built in to defeq it seems like we might be making Lean work harder than is necessary. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict 39/34 Mathlib/Algebra/Homology/ShortComplex/Homology.lean,Mathlib/Algebra/Homology/ShortComplex/RightHomology.lean,Mathlib/CategoryTheory/Idempotents/Basic.lean,Mathlib/CategoryTheory/Limits/HasLimits.lean,Mathlib/CategoryTheory/Limits/Opposites.lean,Mathlib/CategoryTheory/Opposites.lean,Mathlib/CategoryTheory/Sites/CoverLifting.lean,Mathlib/CategoryTheory/Subobject/Comma.lean,Mathlib/CategoryTheory/Triangulated/Opposite.lean,Mathlib/Combinatorics/Quiver/Basic.lean 10 9 ['YaelDillies', 'kim-em', 'leanprover-bot', 'mattrobball'] nobody
313-42770
10 months ago
381-8762
1 year ago
0-0
0 seconds
12934 grunweg
author:grunweg
chore: replace more uses of > or ≥ by < or ≤ These were flagged by the linter in https://github.com/leanprover-community/mathlib4/pull/12879: it is easy to simple avoid > or ≥ in hypotheses or haves. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author help-wanted 41/42 Archive/Imo/Imo1962Q1.lean,Archive/Imo/Imo1988Q6.lean,Archive/Imo/Imo1994Q1.lean,Archive/Imo/Imo2005Q3.lean,Archive/Imo/Imo2006Q3.lean,Archive/Imo/Imo2008Q2.lean,Archive/Imo/Imo2008Q3.lean,Archive/Imo/Imo2019Q4.lean,Archive/Sensitivity.lean,Archive/Wiedijk100Theorems/CubingACube.lean,Mathlib/Tactic/Linarith/Datatypes.lean,test/cancel_denoms.lean,test/congr.lean,test/interval_cases.lean,test/observe.lean 15 11 ['YaelDillies', 'adomani', 'github-actions', 'grunweg', 'jcommelin', 'urkud'] nobody
313-42770
10 months ago
326-52367
10 months ago
1-73101
1 day
12608 eric-wieser
author:eric-wieser
feat: allow `nsmul` / `zsmul` to be omitted again, with a warning --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-meta merge-conflict awaiting-author
label:t-algebra$
118/2 Mathlib.lean,Mathlib/Algebra/Group/Defs.lean,Mathlib/Tactic.lean,Mathlib/Tactic/DefaultFieldLinter.lean,scripts/noshake.json,test/default_field_linter.lean 6 12 ['YaelDillies', 'eric-wieser', 'fpvandoorn', 'github-actions'] nobody
313-42770
10 months ago
362-37834
11 months ago
5-72414
5 days
12588 adomani
author:adomani
remove trailingDegree --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict 1280/979 Mathlib.lean,Mathlib/Algebra/MonoidAlgebra/Basic.lean,Mathlib/Algebra/Polynomial/Degree/Definitions.lean,Mathlib/Algebra/Polynomial/Degree/TrailingDegree.lean,Mathlib/Algebra/Polynomial/Div.lean,Mathlib/Algebra/Polynomial/Mirror.lean,Mathlib/Order/WithBot.lean,Mathlib/Tactic.lean,Mathlib/Tactic/MinMax.lean,Mathlib/Tactic/MinMaxTwo.lean,test/MinMax.lean 11 0 [] nobody
313-42770
10 months ago
401-46346
1 year ago
0-0
0 seconds
12879 grunweg
author:grunweg
feat: port ge_or_gt linter from mathlib3 Code works and is essentially green: next step is to split up into separate PRs. Feedback welcome on whether: - all the test changes are good, or I should simply allow it in more cases - if calc blocks need to be explicitly exempt --- - [ ] depends on: #12933 - [ ] depends on: #12934 - [ ] depends on: #12931 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) tech debt t-linter merge-conflict blocked-by-other-PR 736/319 Archive/Imo/Imo1960Q1.lean,Archive/Imo/Imo1962Q1.lean,Archive/Imo/Imo1988Q6.lean,Archive/Imo/Imo1994Q1.lean,Archive/Imo/Imo2001Q2.lean,Archive/Imo/Imo2005Q3.lean,Archive/Imo/Imo2006Q3.lean,Archive/Imo/Imo2008Q2.lean,Archive/Imo/Imo2008Q3.lean,Archive/Imo/Imo2008Q4.lean,Archive/Imo/Imo2011Q5.lean,Archive/Imo/Imo2019Q4.lean,Archive/Sensitivity.lean,Archive/Wiedijk100Theorems/AreaOfACircle.lean,Archive/Wiedijk100Theorems/BallotProblem.lean,Archive/Wiedijk100Theorems/BirthdayProblem.lean,Archive/Wiedijk100Theorems/CubingACube.lean,Mathlib.lean,Mathlib/Algebra/DualNumber.lean,Mathlib/Algebra/Order/CauSeq/BigOperators.lean,Mathlib/Algebra/Order/Field/Basic.lean,Mathlib/Algebra/Order/Ring/Defs.lean,Mathlib/Algebra/Polynomial/Basic.lean,Mathlib/Algebra/Polynomial/Degree/Definitions.lean,Mathlib/Algebra/Star/CHSH.lean,Mathlib/Analysis/Analytic/Basic.lean,Mathlib/Analysis/Calculus/UniformLimitsDeriv.lean,Mathlib/Analysis/Complex/Hadamard.lean,Mathlib/Analysis/Complex/UpperHalfPlane/Basic.lean,Mathlib/Analysis/InnerProductSpace/Projection.lean,Mathlib/Analysis/Normed/Group/ControlledClosure.lean,Mathlib/Analysis/NormedSpace/MStructure.lean,Mathlib/Analysis/SpecialFunctions/Log/Base.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Basic.lean,Mathlib/Combinatorics/SimpleGraph/DegreeSum.lean,Mathlib/Combinatorics/SimpleGraph/LapMatrix.lean,Mathlib/Computability/AkraBazzi/AkraBazzi.lean,Mathlib/Computability/AkraBazzi/GrowsPolynomially.lean,Mathlib/Data/Complex/Basic.lean,Mathlib/Data/FP/Basic.lean,Mathlib/Data/Finset/Basic.lean,Mathlib/Data/Finset/Fold.lean,Mathlib/Data/Finsupp/Notation.lean,Mathlib/Data/Int/Lemmas.lean,Mathlib/Data/Nat/Dist.lean,Mathlib/Data/Nat/Lattice.lean,Mathlib/Data/Nat/Parity.lean,Mathlib/Data/Nat/Upto.lean,Mathlib/Data/Ordmap/Ordset.lean,Mathlib/Data/PNat/Basic.lean,Mathlib/Data/UInt.lean,Mathlib/GroupTheory/Coxeter/Length.lean,Mathlib/MeasureTheory/Constructions/Polish.lean,Mathlib/MeasureTheory/Covering/Besicovitch.lean,Mathlib/MeasureTheory/Covering/Vitali.lean,Mathlib/MeasureTheory/Covering/VitaliFamily.lean,Mathlib/MeasureTheory/Integral/Layercake.lean,Mathlib/NumberTheory/LegendreSymbol/JacobiSymbol.lean,Mathlib/NumberTheory/Padics/Hensel.lean,Mathlib/NumberTheory/Padics/PadicNorm.lean,Mathlib/NumberTheory/PellMatiyasevic.lean,Mathlib/NumberTheory/Rayleigh.lean,Mathlib/Order/Filter/AtTopBot.lean,Mathlib/Probability/Process/Stopping.lean,Mathlib/RingTheory/Adjoin/Basic.lean,Mathlib/RingTheory/Polynomial/Basic.lean,Mathlib/SetTheory/Ordinal/Notation.lean,Mathlib/Tactic.lean,Mathlib/Tactic/CancelDenoms/Core.lean,Mathlib/Tactic/Common.lean,Mathlib/Tactic/IntervalCases.lean,Mathlib/Tactic/Linarith/Datatypes.lean,Mathlib/Tactic/Linarith/Lemmas.lean,Mathlib/Tactic/Linarith/Oracle/FourierMotzkin.lean,Mathlib/Tactic/Linter/GeOrGt.lean,Mathlib/Tactic/Linter/Style.lean,Mathlib/Tactic/NormNum/GCD.lean,Mathlib/Tactic/NormNum/Inv.lean,Mathlib/Tactic/Ring/Basic.lean,Mathlib/Topology/Category/Profinite/Nobeling.lean,Mathlib/Topology/ContinuousFunction/Bounded.lean,Mathlib/Topology/MetricSpace/CauSeqFilter.lean,Mathlib/Topology/MetricSpace/Cauchy.lean,Mathlib/Topology/MetricSpace/Closeds.lean,Mathlib/Topology/Sequences.lean,scripts/lint-style.py,test/Explode.lean,test/GCongr/inequalities.lean,test/GeOrGt.lean,test/LibrarySearch/IsCompact.lean,test/LibrarySearch/basic.lean,test/Recall.lean,test/Rify.lean,test/Use.lean,test/cancel_denoms.lean,test/congr.lean,test/delabLinearIndependent.lean,test/delaborators.lean,test/interval_cases.lean,test/linarith.lean 109 3 ['github-actions', 'grunweg', 'leanprover-community-mathlib4-bot'] nobody
313-42770
10 months ago
335-23470
11 months ago
0-15202
4 hours
12473 adomani
author:adomani
first translations --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict 424/265 Mathlib.lean,Mathlib/Order/Lattice.lean,Mathlib/Order/WithBot.lean,Mathlib/Tactic.lean,Mathlib/Tactic/MinMax.lean 5 0 [] nobody
313-42770
10 months ago
383-42913
1 year ago
0-0
0 seconds
12773 apnelson1
author:apnelson1
feat(Combinatorics/HypergraphRamsey): Ramsey's theorem for hypergraphs This PR is an unborked version of #12167, which had some bad merge conflicts. We prove Ramsey's theorem for infinite hypergraphs: for any colouring of the k-subsets of an infinite set S with a finite set of colours, there is an infinite subset T of S whose k-subsets all have the same colour. The finite versions will follow from compactness techniques, but aren't included here. (#12273 is the first step for this). The proof encodes k-subsets as order-embeddings from Fin k rather than as Finsets, as this makes things more convenient, and should extend better to generalizations like the canonical Ramsey theorem. This requires a small amount of API to be added, including some simple instances for `OrderEmbedding`. We also require a result saying that there is a list of all k-subsets of Nat for which the sequence of largest elements is monotone. We do this by adding some new material in Order.Extension.Linear, which has more general applications. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics merge-conflict 623/2 Mathlib.lean,Mathlib/Combinatorics/HypergraphRamsey.lean,Mathlib/Data/Finset/Sort.lean,Mathlib/Order/Extension/Linear.lean,Mathlib/Order/Hom/Basic.lean,Mathlib/Order/Interval/Finset/Defs.lean,Mathlib/Order/OrderIsoNat.lean,Mathlib/Order/RelClasses.lean,lean-toolchain 9 3 ['github-actions', 'loefflerd'] nobody
313-42770
10 months ago
335-23470
11 months ago
39-66196
39 days
12679 MichaelStollBayreuth
author:MichaelStollBayreuth
perf(NumberTheory/RamificationInertia): speed up slow file A repetition of the earlier experiment at [#12412](https://github.com/leanprover-community/mathlib4/pull/12412) with Lean 4.8.0-rc1. This time, I tried not to introduce local instances if possible, but instead to tweak instance priorities. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP 57/14 Mathlib/NumberTheory/RamificationInertia.lean 1 3 ['MichaelStollBayreuth', 'github-actions', 'leanprover-bot'] nobody
313-42770
10 months ago
371-1915
1 year ago
0-0
0 seconds
12637 adomani
author:adomani
translation: MonoidAlgebra to AddMonoidAlgebra [Zulip discussion](https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/merge.20Add-MonoidAlgebra) * #12646 was found as a consequence of unification. * #12659 the typo `single 1 1` for `single 0 1`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-meta merge-conflict
label:t-algebra$
615/986 Mathlib.lean,Mathlib/Algebra/MonoidAlgebra/Basic.lean,Mathlib/Algebra/MonoidAlgebra/Division.lean,Mathlib/Algebra/MvPolynomial/Basic.lean,Mathlib/Tactic.lean,Mathlib/Tactic/MinMaxTwo.lean,scripts/noshake.json 7 0 [] nobody
313-42770
10 months ago
335-23470
11 months ago
0-0
0 seconds
12416 adomani
author:adomani
chore: remove some cdots --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict 3830/3239 Archive/Imo/Imo1972Q5.lean,Archive/Imo/Imo2006Q5.lean,Archive/Imo/Imo2008Q2.lean,Archive/Imo/Imo2021Q1.lean,Archive/Wiedijk100Theorems/AbelRuffini.lean,Archive/Wiedijk100Theorems/BallotProblem.lean,Archive/Wiedijk100Theorems/BirthdayProblem.lean,Archive/Wiedijk100Theorems/BuffonsNeedle.lean,Archive/Wiedijk100Theorems/CubingACube.lean,Archive/Wiedijk100Theorems/FriendshipGraphs.lean,Archive/Wiedijk100Theorems/Partition.lean,Counterexamples/Cyclotomic105.lean,Counterexamples/DirectSumIsInternal.lean,Mathlib.lean,Mathlib/Algebra/Algebra/Spectrum.lean,Mathlib/Algebra/BigOperators/Finprod.lean,Mathlib/Algebra/BigOperators/List/Basic.lean,Mathlib/Algebra/Category/GroupCat/Colimits.lean,Mathlib/Algebra/Category/ModuleCat/Images.lean,Mathlib/Algebra/Category/Ring/Constructions.lean,Mathlib/Algebra/CharP/Quotient.lean,Mathlib/Algebra/ContinuedFractions/Computation/Approximations.lean,Mathlib/Algebra/DirectLimit.lean,Mathlib/Algebra/DirectSum/Internal.lean,Mathlib/Algebra/GCDMonoid/Finset.lean,Mathlib/Algebra/GeomSum.lean,Mathlib/Algebra/Group/UniqueProds.lean,Mathlib/Algebra/GroupPower/Order.lean,Mathlib/Algebra/GroupWithZero/WithZero.lean,Mathlib/Algebra/Homology/Exact.lean,Mathlib/Algebra/Homology/HomotopyCategory/HomComplex.lean,Mathlib/Algebra/Homology/HomotopyCategory/Triangulated.lean,Mathlib/Algebra/Homology/LocalCohomology.lean,Mathlib/Algebra/Homology/TotalComplex.lean,Mathlib/Algebra/Lie/DirectSum.lean,Mathlib/Algebra/Lie/IdealOperations.lean,Mathlib/Algebra/Lie/Nilpotent.lean,Mathlib/Algebra/Lie/Weights/Basic.lean,Mathlib/Algebra/Module/DedekindDomain.lean,Mathlib/Algebra/Module/LinearMap/End.lean,Mathlib/Algebra/Module/LocalizedModule.lean,Mathlib/Algebra/Module/PID.lean,Mathlib/Algebra/Module/Submodule/Bilinear.lean,Mathlib/Algebra/Module/Torsion.lean,Mathlib/Algebra/Module/Zlattice/Basic.lean,Mathlib/Algebra/MonoidAlgebra/Basic.lean,Mathlib/Algebra/MonoidAlgebra/Degree.lean,Mathlib/Algebra/MonoidAlgebra/Ideal.lean,Mathlib/Algebra/MvPolynomial/Variables.lean,Mathlib/Algebra/Order/Archimedean.lean,Mathlib/Algebra/Order/BigOperators/Group/List.lean,Mathlib/Algebra/Order/CauSeq/BigOperators.lean,Mathlib/Algebra/Order/CompleteField.lean,Mathlib/Algebra/Order/Field/Basic.lean,Mathlib/Algebra/Order/Group/Abs.lean,Mathlib/Algebra/Order/Group/Int.lean,Mathlib/Algebra/Order/Group/MinMax.lean,Mathlib/Algebra/Order/Interval/Basic.lean,Mathlib/Algebra/Order/Pointwise.lean,Mathlib/Algebra/Order/Sub/Defs.lean,Mathlib/Algebra/Polynomial/BigOperators.lean,Mathlib/Algebra/Polynomial/Degree/Definitions.lean,Mathlib/Algebra/Polynomial/Derivative.lean,Mathlib/Algebra/Polynomial/Div.lean,Mathlib/Algebra/Polynomial/FieldDivision.lean,Mathlib/Algebra/Polynomial/Module/Basic.lean,Mathlib/Algebra/Polynomial/PartialFractions.lean,Mathlib/Algebra/Polynomial/Reverse.lean,Mathlib/Algebra/Polynomial/RingDivision.lean,Mathlib/Algebra/Polynomial/UnitTrinomial.lean,Mathlib/Algebra/Quandle.lean,Mathlib/Algebra/Quaternion.lean,Mathlib/AlgebraicGeometry/AffineScheme.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Affine.lean,Mathlib/AlgebraicGeometry/FunctionField.lean,Mathlib/AlgebraicGeometry/Gluing.lean,Mathlib/AlgebraicGeometry/Morphisms/Basic.lean,Mathlib/AlgebraicGeometry/Morphisms/QuasiCompact.lean,Mathlib/AlgebraicGeometry/Morphisms/QuasiSeparated.lean,Mathlib/AlgebraicGeometry/Morphisms/RingHomProperties.lean,Mathlib/AlgebraicGeometry/OpenImmersion.lean,Mathlib/AlgebraicGeometry/ProjectiveSpectrum/Scheme.lean,Mathlib/AlgebraicGeometry/Properties.lean,Mathlib/AlgebraicGeometry/Pullbacks.lean,Mathlib/AlgebraicGeometry/StructureSheaf.lean,Mathlib/AlgebraicTopology/SimplexCategory.lean,Mathlib/AlgebraicTopology/SplitSimplicialObject.lean,Mathlib/Analysis/Analytic/Composition.lean,Mathlib/Analysis/Analytic/IsolatedZeros.lean,Mathlib/Analysis/BoundedVariation.lean,Mathlib/Analysis/BoxIntegral/Box/Basic.lean,Mathlib/Analysis/BoxIntegral/Partition/Basic.lean,Mathlib/Analysis/Calculus/ContDiff/Basic.lean,Mathlib/Analysis/Calculus/Deriv/Slope.lean,Mathlib/Analysis/Calculus/FDeriv/Basic.lean,Mathlib/Analysis/Calculus/FDeriv/Extend.lean,Mathlib/Analysis/Calculus/InverseFunctionTheorem/ApproximatesLinearOn.lean,Mathlib/Analysis/Calculus/LocalExtr/Basic.lean,Mathlib/Analysis/Calculus/ParametricIntegral.lean,Mathlib/Analysis/Calculus/TangentCone.lean 608 0 [] nobody
313-42770
10 months ago
405-44768
1 year ago
0-0
0 seconds
12192 Ruben-VandeVelde
author:Ruben-VandeVelde
feat: generalize isLittleO_const_id_atTop/atBot From PNT+. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis merge-conflict awaiting-author 10/4 Mathlib/Analysis/Asymptotics/Asymptotics.lean 1 6 ['Ruben-VandeVelde', 'llllvvuu', 'urkud'] nobody
313-42769
10 months ago
325-20636
10 months ago
1-21749
1 day
11575 ScottCarnahan
author:ScottCarnahan
feat (RingTheory/HahnSeries/Addition): Lemmas on leading terms The main result of this PR is that when the exponent set is linearly ordered, then removing the leading term in a Hahn series `x` yields a Hahn series `y` that is, if nonzero, of strictly higher order. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict WIP
label:t-algebra$
39/0 Mathlib/RingTheory/HahnSeries/Addition.lean 1 0 [] nobody
313-42769
10 months ago
333-81932
10 months ago
10-75677
10 days
11617 urkud
author:urkud
refactor(Finset): redefine Finset.diag, review API Redefine `Finset.diag` using `Finset.map`. The new definition doesn't rely on `DecidableEq` and is much more computationally efficient. Also review API and golf proofs here and there. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-logic merge-conflict awaiting-author 187/181 Archive/Imo/Imo1998Q2.lean,Mathlib.lean,Mathlib/Algebra/BigOperators/Basic.lean,Mathlib/Combinatorics/SimpleGraph/Regularity/Energy.lean,Mathlib/Combinatorics/SimpleGraph/Regularity/Increment.lean,Mathlib/Combinatorics/SimpleGraph/Regularity/Uniform.lean,Mathlib/Data/Finset/Diag.lean,Mathlib/Data/Finset/Image.lean,Mathlib/Data/Finset/Prod.lean,Mathlib/Data/Set/Image.lean,Mathlib/Data/Set/Prod.lean,Mathlib/Data/Sym/Card.lean,Mathlib/Data/Sym/Sym2.lean 13 7 ['YaelDillies', 'eric-wieser', 'urkud'] nobody
313-42769
10 months ago
435-80899
1 year ago
1-12270
1 day
12292 AntoineChambert-Loir
author:AntoineChambert-Loir
feat(Mathlib.RingTheory.TensorProduct.MonoidAlgebra) : tensor product of a monoid algebra * `MonoidAlgebra.rTensorAlgEquiv`: the tensor product of `MonoidAlgebra M α` with `N` is `R`-linearly equivalent to `MonoidAlgebra (M ⊗[R] N) α` * `MonoidAlgebra.scalarRTensorAlgEquiv`, the tensor product of `MonoidAlgebra R α` with `N` is `R`-linearly equivalent to `MonoidAlgebra N α` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict WIP
label:t-algebra$
447/0 Mathlib.lean,Mathlib/Data/Finsupp/Defs.lean,Mathlib/RingTheory/TensorProduct/MonoidAlgebra.lean 3 23 ['AntoineChambert-Loir', 'eric-wieser', 'github-actions'] nobody
313-42769
10 months ago
335-23470
11 months ago
6-28213
6 days
12181 adomani
author:adomani
lint also `let` vs `have` This PR is symmetrical to #12157: here we lint for non-`Type`-valued `let`s. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict 797/544 Archive/Imo/Imo1962Q1.lean,Archive/Wiedijk100Theorems/CubingACube.lean,Archive/Wiedijk100Theorems/FriendshipGraphs.lean,Mathlib.lean,Mathlib/Algebra/Algebra/Tower.lean,Mathlib/Algebra/BigOperators/Basic.lean,Mathlib/Algebra/DirectLimit.lean,Mathlib/Algebra/Group/UniqueProds.lean,Mathlib/Algebra/Homology/HomologicalComplexBiprod.lean,Mathlib/Algebra/Homology/HomologySequence.lean,Mathlib/Algebra/Homology/HomotopyCategory/Pretriangulated.lean,Mathlib/Algebra/Homology/Localization.lean,Mathlib/Algebra/Homology/ShortComplex/Abelian.lean,Mathlib/Algebra/Homology/ShortComplex/ConcreteCategory.lean,Mathlib/Algebra/Homology/ShortComplex/Exact.lean,Mathlib/Algebra/Homology/ShortComplex/ExactFunctor.lean,Mathlib/Algebra/Homology/ShortComplex/Homology.lean,Mathlib/Algebra/Homology/ShortComplex/LeftHomology.lean,Mathlib/Algebra/Homology/ShortComplex/Linear.lean,Mathlib/Algebra/Homology/ShortComplex/Preadditive.lean,Mathlib/Algebra/Homology/ShortComplex/PreservesHomology.lean,Mathlib/Algebra/Homology/ShortComplex/QuasiIso.lean,Mathlib/Algebra/Homology/ShortComplex/RightHomology.lean,Mathlib/Algebra/Lie/Engel.lean,Mathlib/Algebra/Lie/Killing.lean,Mathlib/Algebra/Module/PID.lean,Mathlib/Algebra/Module/Submodule/Localization.lean,Mathlib/Algebra/Module/Zlattice.lean,Mathlib/Algebra/MonoidAlgebra/Grading.lean,Mathlib/Algebra/MvPolynomial/Equiv.lean,Mathlib/Algebra/Order/CauSeq/Basic.lean,Mathlib/Algebra/Polynomial/FieldDivision.lean,Mathlib/Algebra/Polynomial/RingDivision.lean,Mathlib/AlgebraicGeometry/Morphisms/QuasiCompact.lean,Mathlib/AlgebraicGeometry/Morphisms/QuasiSeparated.lean,Mathlib/AlgebraicGeometry/ProjectiveSpectrum/Scheme.lean,Mathlib/AlgebraicGeometry/Pullbacks.lean,Mathlib/AlgebraicGeometry/StructureSheaf.lean,Mathlib/AlgebraicTopology/DoldKan/Homotopies.lean,Mathlib/Analysis/Calculus/ContDiff/Basic.lean,Mathlib/Analysis/Calculus/ContDiff/Bounds.lean,Mathlib/Analysis/Calculus/FDeriv/Comp.lean,Mathlib/Analysis/Calculus/Rademacher.lean,Mathlib/Analysis/Complex/Tietze.lean,Mathlib/Analysis/Convex/Between.lean,Mathlib/Analysis/Convolution.lean,Mathlib/Analysis/Fourier/RiemannLebesgueLemma.lean,Mathlib/Analysis/InnerProductSpace/GramSchmidtOrtho.lean,Mathlib/Analysis/InnerProductSpace/PiL2.lean,Mathlib/Analysis/InnerProductSpace/Rayleigh.lean,Mathlib/Analysis/NormedSpace/ContinuousAffineMap.lean,Mathlib/Analysis/NormedSpace/OperatorNorm/Completeness.lean,Mathlib/Analysis/NormedSpace/Spectrum.lean,Mathlib/Analysis/SpecialFunctions/Integrals.lean,Mathlib/CategoryTheory/Abelian/Basic.lean,Mathlib/CategoryTheory/Abelian/Exact.lean,Mathlib/CategoryTheory/Abelian/Pseudoelements.lean,Mathlib/CategoryTheory/Abelian/Transfer.lean,Mathlib/CategoryTheory/Adhesive.lean,Mathlib/CategoryTheory/Closed/Cartesian.lean,Mathlib/CategoryTheory/Closed/Monoidal.lean,Mathlib/CategoryTheory/Comma/Arrow.lean,Mathlib/CategoryTheory/EffectiveEpi/Extensive.lean,Mathlib/CategoryTheory/Extensive.lean,Mathlib/CategoryTheory/Functor/EpiMono.lean,Mathlib/CategoryTheory/Functor/KanExtension/Basic.lean,Mathlib/CategoryTheory/Galois/Basic.lean,Mathlib/CategoryTheory/Galois/Decomposition.lean,Mathlib/CategoryTheory/Galois/Examples.lean,Mathlib/CategoryTheory/GradedObject/Trifunctor.lean,Mathlib/CategoryTheory/IsConnected.lean,Mathlib/CategoryTheory/Limits/ConcreteCategory.lean,Mathlib/CategoryTheory/Limits/Constructions/EpiMono.lean,Mathlib/CategoryTheory/Limits/Constructions/WeaklyInitial.lean,Mathlib/CategoryTheory/Limits/FilteredColimitCommutesFiniteLimit.lean,Mathlib/CategoryTheory/Limits/Final.lean,Mathlib/CategoryTheory/Limits/FintypeCat.lean,Mathlib/CategoryTheory/Limits/Fubini.lean,Mathlib/CategoryTheory/Limits/IsLimit.lean,Mathlib/CategoryTheory/Limits/Preserves/Basic.lean,Mathlib/CategoryTheory/Limits/Shapes/FiniteLimits.lean,Mathlib/CategoryTheory/Limits/VanKampen.lean,Mathlib/CategoryTheory/Localization/LocalizerMorphism.lean,Mathlib/CategoryTheory/Localization/Pi.lean,Mathlib/CategoryTheory/Localization/Resolution.lean,Mathlib/CategoryTheory/Monad/Monadicity.lean,Mathlib/CategoryTheory/PUnit.lean,Mathlib/CategoryTheory/Sites/Coherent/CoherentSheaves.lean,Mathlib/CategoryTheory/Sites/Coherent/RegularSheaves.lean,Mathlib/CategoryTheory/Sites/Coverage.lean,Mathlib/CategoryTheory/Sites/LeftExact.lean,Mathlib/CategoryTheory/Sites/Preserves.lean,Mathlib/CategoryTheory/Sites/Pullback.lean,Mathlib/CategoryTheory/Sites/Sheaf.lean,Mathlib/CategoryTheory/Triangulated/Pretriangulated.lean,Mathlib/Combinatorics/Colex.lean,Mathlib/Combinatorics/SetFamily/Kleitman.lean,Mathlib/Combinatorics/SimpleGraph/Clique.lean,Mathlib/Combinatorics/SimpleGraph/Coloring.lean,Mathlib/Combinatorics/SimpleGraph/Connectivity.lean 271 0 [] nobody
313-42769
10 months ago
418-33976
1 year ago
0-0
0 seconds
11100 eric-wieser
author:eric-wieser
feat(CategoryTheory/Limits): add `Functor.mapBinaryBiconeInv` --- - [ ] depends on: #11130 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) It's tempting to try to prove something like ```lean theorem Functor.mapBinaryBiconeInv_toCone [Limits.HasZeroMorphisms C] [Limits.HasZeroMorphisms D] (e : D ⥤ C) [IsEquivalence e] {X Y : D} (b : BinaryBicone (e.obj X) (e.obj Y)) : (e.mapBinaryBiconeInv b).toCone = (e.mapConeInv <| (Cones.postcompose (pairComp X Y e).symm.hom).obj b.toCone) := by simp sorry theorem Functor.mapBinaryBiconeInv_toCocone [Limits.HasZeroMorphisms C] [Limits.HasZeroMorphisms D] (e : D ⥤ C) [IsEquivalence e] {X Y : D} (b : BinaryBicone (e.obj X) (e.obj Y)) : (e.mapBinaryBiconeInv b).toCocone = (e.mapCoconeInv <| (Cocones.precompose (pairComp X Y e).hom).obj b.toCocone) := by sorry ``` but maybe equality is evil here t-category-theory awaiting-CI merge-conflict 52/0 Mathlib/CategoryTheory/Adjunction/Basic.lean,Mathlib/CategoryTheory/Equivalence.lean,Mathlib/CategoryTheory/Limits/Preserves/Shapes/Biproducts.lean 3 6 ['TwoFX', 'eric-wieser', 'leanprover-community-mathlib4-bot'] nobody
313-42768
10 months ago
335-23470
11 months ago
0-0
0 seconds
10845 Shamrock-Frost
author:Shamrock-Frost
Refactor: Make MonoidalFunctor carry the data of an inverse We change the definition of a strong monoidal functor from a lax monoidal functor for which the unitor and tensorator are `IsIso` to a lax monoidal functor with the data of inverses for the unitor and tensorator. This requires fixing a lot of knock on effects. --- This is a **draft PR**. I would like to talk with people on zulip before merging it, and plan ahead to when we have oplax/colax monoidal functors as well. I'm not sure the approach I took here where `MonoidalFunctor` inherits from `LaxMonoidalFunctor` is a good choice if we want to be lax/oplax symmetric. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory RFC merge-conflict WIP 3799/1589 Mathlib/Algebra/Category/ModuleCat/Adjunctions.lean,Mathlib/Algebra/Homology/HomotopyCategory/DegreewiseSplit.lean,Mathlib/CategoryTheory/Adjunction/Basic.lean,Mathlib/CategoryTheory/Adjunction/Mates.lean,Mathlib/CategoryTheory/Adjunction/Opposites.lean,Mathlib/CategoryTheory/Adjunction/Prod.lean,Mathlib/CategoryTheory/Adjunction/Whiskering.lean,Mathlib/CategoryTheory/Bicategory/End.lean,Mathlib/CategoryTheory/Bicategory/SingleObj.lean,Mathlib/CategoryTheory/CatCommSq.lean,Mathlib/CategoryTheory/CatSquares.lean,Mathlib/CategoryTheory/Enriched/Basic.lean,Mathlib/CategoryTheory/Equivalence.lean,Mathlib/CategoryTheory/Iso.lean,Mathlib/CategoryTheory/Monoidal/Adjunction.lean,Mathlib/CategoryTheory/Monoidal/Braided.lean,Mathlib/CategoryTheory/Monoidal/Category.lean,Mathlib/CategoryTheory/Monoidal/Center.lean,Mathlib/CategoryTheory/Monoidal/CommMon_.lean,Mathlib/CategoryTheory/Monoidal/Discrete.lean,Mathlib/CategoryTheory/Monoidal/End.lean,Mathlib/CategoryTheory/Monoidal/Free/Basic.lean,Mathlib/CategoryTheory/Monoidal/Functor.lean,Mathlib/CategoryTheory/Monoidal/Limits.lean,Mathlib/CategoryTheory/Monoidal/Mon_.lean,Mathlib/CategoryTheory/Monoidal/NaturalTransformation.lean,Mathlib/CategoryTheory/Monoidal/Opposite.lean,Mathlib/CategoryTheory/Monoidal/Rigid/FunctorCategory.lean,Mathlib/CategoryTheory/Monoidal/Rigid/OfEquivalence.lean,Mathlib/CategoryTheory/Monoidal/Subcategory.lean,Mathlib/CategoryTheory/Monoidal/Transport.lean,Mathlib/CategoryTheory/Monoidal/Types/Basic.lean,Mathlib/CategoryTheory/Opposites.lean,Mathlib/CategoryTheory/Products/Associator.lean,Mathlib/CategoryTheory/Products/Basic.lean,Mathlib/CategoryTheory/Shift/Basic.lean,Mathlib/CategoryTheory/Shift/Pullback.lean,Mathlib/CategoryTheory/Whiskering.lean,Mathlib/RepresentationTheory/Action/Monoidal.lean,Mathlib/RepresentationTheory/GroupCohomology/Resolution.lean,Mathlib/RepresentationTheory/Rep.lean 41 7 ['Shamrock-Frost', 'joelriou'] nobody
313-42768
10 months ago
468-67301
1 year ago
0-0
0 seconds
11021 jstoobysmith
author:jstoobysmith
feat(AlgebraicTopology) : add join of augmented SSets This pull-request adds the definition of the join of augmented SSets defined as contravariant functors from `WithInitial SimplexCategory` to `Type u`. In addition it shows that the join of two standard augmented SSets is again an augmented SSets. From this the definition of the join of simplicial sets should follow easily. To aid the above theory, an api for `WithInitial SimplexCategory` has been created, with the notion of the `join` and `split` (forming a sort of inverse to join) of objects in this category are defined. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-category-theory merge-conflict WIP 2137/1 .gitignore,Mathlib.lean,Mathlib/AlgebraicTopology/Join.lean,Mathlib/AlgebraicTopology/SimplexCategory.lean,Mathlib/AlgebraicTopology/SimplexCategoryWithInitial.lean,Mathlib/AlgebraicTopology/SimplicialSet.lean 6 47 ['github-actions', 'jcommelin'] nobody
313-42768
10 months ago
369-37814
1 year ago
1-20125
1 day
10842 mcdoll
author:mcdoll
chore: simplify proofs using new positivity extensions and tests --- - [x] depends on: #10661 - [ ] depends on: #10796 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR WIP 98/50 Mathlib/Analysis/Convolution.lean,Mathlib/Analysis/SpecialFunctions/Gaussian.lean,Mathlib/MeasureTheory/Covering/Differentiation.lean,Mathlib/MeasureTheory/Function/ConditionalExpectation/CondexpL1.lean,Mathlib/MeasureTheory/Function/ConditionalExpectation/Real.lean,Mathlib/MeasureTheory/Function/ConditionalExpectation/Unique.lean,Mathlib/MeasureTheory/Function/ContinuousMapDense.lean,Mathlib/MeasureTheory/Integral/Bochner.lean,Mathlib/MeasureTheory/Measure/Tilted.lean,Mathlib/Probability/Martingale/Upcrossing.lean,Mathlib/Probability/Moments.lean,Mathlib/Probability/Variance.lean,Mathlib/Tactic/Positivity/Core.lean,test/positivity.lean 14 1 ['leanprover-community-mathlib4-bot'] nobody
313-42768
10 months ago
377-45989
1 year ago
0-0
0 seconds
10126 Multramate
author:Multramate
feat(GroupTheory/GroupAction/Basic): define homomorphisms of fixed subgroups induced by homomorphisms of groups --- - [ ] depends on: #10043 - [ ] depends on: #10113 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict blocked-by-other-PR
label:t-algebra$
81/12 Mathlib/GroupTheory/GroupAction/Basic.lean,Mathlib/GroupTheory/Subgroup/Basic.lean,Mathlib/GroupTheory/Submonoid/Operations.lean 3 1 ['leanprover-community-mathlib4-bot'] nobody
313-42768
10 months ago
335-23470
11 months ago
0-0
0 seconds
10113 Multramate
author:Multramate
feat(GroupTheory/Submonoid/Operations): define homomorphisms of subgroups induced by homomorphisms of groups --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict awaiting-author
label:t-algebra$
29/6 Mathlib/GroupTheory/Subgroup/Basic.lean,Mathlib/GroupTheory/Submonoid/Operations.lean 2 1 ['ocfnash'] ocfnash
assignee:ocfnash
313-42768
10 months ago
402-19069
1 year ago
22-57316
22 days
10521 eric-wieser
author:eric-wieser
chore: generalize `IsBoundedLinearMap` to modules Most of the lemmas don't actually need the normed on the scalars at all. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis merge-conflict awaiting-author 58/42 Mathlib/Analysis/NormedSpace/BoundedLinearMaps.lean 1 3 ['github-actions', 'j-loreaux', 'urkud'] nobody
313-42768
10 months ago
420-56830
1 year ago
1-29105
1 day
10024 ADedecker
author:ADedecker
feat: rename `connectedComponentOfOne` to `identityComponent`, prove that it is normal and open --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology awaiting-CI merge-conflict 58/24 Mathlib/FieldTheory/AbsoluteGaloisGroup.lean,Mathlib/Topology/Algebra/Group/Basic.lean,Mathlib/Topology/Algebra/Group/TopologicalAbelianization.lean,Mathlib/Topology/Algebra/OpenSubgroup.lean,Mathlib/Topology/Connected/Basic.lean 5 0 [] nobody
313-42768
10 months ago
325-21225
10 months ago
0-832
13 minutes
10444 urkud
author:urkud
doc(IsROrC): expand the docstring --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis merge-conflict awaiting-author documentation 34/0 Mathlib/Data/IsROrC/Basic.lean 1 9 ['eric-wieser', 'kbuzzard', 'urkud'] nobody
313-42768
10 months ago
438-28660
1 year ago
1-62352
1 day
10142 Multramate
author:Multramate
feat(AlgebraicGeometry/EllipticCurve/Group): compute range of baseChange --- - [x] depends on: #9744 - [x] depends on: #10043 - [ ] depends on: #10113 - [ ] depends on: #10126 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebraic-geometry t-number-theory merge-conflict blocked-by-other-PR 421/212 Mathlib/AlgebraicGeometry/EllipticCurve/Affine.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Group.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Weierstrass.lean,Mathlib/GroupTheory/GroupAction/Basic.lean,Mathlib/GroupTheory/Subgroup/Basic.lean,Mathlib/GroupTheory/Submonoid/Operations.lean 6 3 ['Multramate', 'alreadydone', 'leanprover-community-mathlib4-bot'] nobody
313-42768
10 months ago
335-23470
11 months ago
0-0
0 seconds
10721 urkud
author:urkud
feat(Order/FunLike): define `PointwiseLE` - introduce a mixin class `DFunLike.PointwiseLE`, use it to define `DFunLike.instPartialOrder`; - add a generic `DFunLike.orderEmbeddingCoe` - add `DFunLike.PointwiseLE` instances here and there. With this refactor and #13022, I'm going to generalize lemmas like `MeasureTheory.ae_mono` to `OuterMeasureClass`. --- - [x] depends on: #12983 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-logic t-order merge-conflict 123/50 Mathlib.lean,Mathlib/Algebra/Order/Hom/Ring.lean,Mathlib/Data/DFinsupp/Order.lean,Mathlib/Data/Finsupp/Order.lean,Mathlib/Data/FunLike/Basic.lean,Mathlib/Dynamics/Circle/RotationNumber/TranslationNumber.lean,Mathlib/GroupTheory/Congruence.lean,Mathlib/Order/FunLike.lean,Mathlib/Order/Heyting/Hom.lean,Mathlib/Order/Hom/Basic.lean,Mathlib/Order/Hom/Bounded.lean,Mathlib/Order/Hom/CompleteLattice.lean,Mathlib/Topology/Order/Hom/Basic.lean 13 48 ['YaelDillies', 'dupuisf', 'leanprover-community-mathlib4-bot', 'urkud'] nobody
313-42768
10 months ago
335-23470
11 months ago
64-12826
64 days
10594 lecopivo
author:lecopivo
feat: `fun_trans` function transformation tactic e.g. for computing derivatives feat: `fun_trans` function transformation tactic e.g. for computing derivatives Function transformation tactic/simproc. For example it can be used for computing derivatives. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta merge-conflict WIP 1819/56 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/FunProp/Core.lean,Mathlib/Tactic/FunProp/Decl.lean,Mathlib/Tactic/FunProp/Elab.lean,Mathlib/Tactic/FunProp/FunctionData.lean,Mathlib/Tactic/FunProp/MorExt.lean,Mathlib/Tactic/FunProp/Theorems.lean,Mathlib/Tactic/FunTrans/Attr.lean,Mathlib/Tactic/FunTrans/Core.lean,Mathlib/Tactic/FunTrans/Decl.lean,Mathlib/Tactic/FunTrans/Elab.lean,Mathlib/Tactic/FunTrans/Theorems.lean,Mathlib/Tactic/FunTrans/Types.lean,test/fun_prop2.lean,test/fun_prop_dev.lean,test/fun_trans_dev.lean 17 11 ['github-actions'] nobody
313-42768
10 months ago
374-66427
1 year ago
0-0
0 seconds
8616 eric-wieser
author:eric-wieser
feat(Algebra/FreeAlgebra): add right action and `IsCentralScalar` --- - [ ] depends on: #8652 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra awaiting-CI merge-conflict
label:t-algebra$
30/8 Mathlib/Algebra/FreeAlgebra.lean 1 1 ['leanprover-community-mathlib4-bot'] nobody
313-42767
10 months ago
335-23470
11 months ago
0-0
0 seconds
8519 eric-wieser
author:eric-wieser
refactor(LinearAlgebra/TensorProduct): golf using `liftAddHom` This new `TensorProduct.liftAddHom` doesn't require bilinearity, only that scalar multiplication can be moved between the arguments. While in theory we only need the `AddMonoidHom` version as it offers exactly the same generality, we first provide an unbundled `liftFun` as this seems to give a sizeable performance boost if used in downstream `lift` variants. --- - [x] depends on: #8571 - [x] depends on: #8584 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict awaiting-author
label:t-algebra$
53/50 Mathlib/Algebra/Category/AlgebraCat/Monoidal.lean,Mathlib/LinearAlgebra/TensorProduct.lean,Mathlib/LinearAlgebra/TensorProduct/Tower.lean 3 28 ['bustercopley', 'eric-wieser', 'jcommelin', 'jjaassoonn', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'mathlib-bors'] nobody
313-42767
10 months ago
462-15082
1 year ago
5-6524
5 days
8788 FMLJohn
author:FMLJohn
feat(Algebra/Module/GradeZeroModule): if `A` is a graded semiring and `M` is a graded `A`-module, then each grade of `M` is a module over the 0-th grade of `A`. --- - [ ] depends on: #8187 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict
label:t-algebra$
237/4 Mathlib.lean,Mathlib/Algebra/DirectSum/Internal.lean,Mathlib/Algebra/GradedMonoid.lean,Mathlib/Algebra/Module/GradeZeroModule.lean,Mathlib/RingTheory/GradedAlgebra/Basic.lean,Mathlib/RingTheory/GradedAlgebra/Noetherian.lean 6 4 ['FMLJohn', 'github-actions', 'leanprover-community-mathlib4-bot'] nobody
313-42767
10 months ago
347-30669
11 months ago
0-0
0 seconds
8906 jjaassoonn
author:jjaassoonn
feat: add some missing lemmas about linear algebra --- - [ ] depends on: #8905 [lifting injective modules to higher universe] [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict awaiting-author
label:t-algebra$
45/1 Mathlib/Algebra/Category/ModuleCat/Basic.lean,Mathlib/Algebra/Module/Injective.lean,Mathlib/LinearAlgebra/Basic.lean,Mathlib/LinearAlgebra/BilinearMap.lean 4 21 ['AntoineChambert-Loir', 'alreadydone', 'jjaassoonn', 'leanprover-community-mathlib4-bot'] nobody
313-42767
10 months ago
414-78896
1 year ago
0-0
0 seconds
8961 eric-wieser
author:eric-wieser
refactor: use the coinduced topology on ULift --- - [x] depends on: #8958 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-CI merge-conflict please-adopt awaiting-author 46/14 Mathlib/Analysis/Normed/Group/Basic.lean,Mathlib/Topology/Bornology/Constructions.lean,Mathlib/Topology/Constructions.lean 3 6 ['eric-wieser', 'github-actions', 'leanprover-community-mathlib4-bot', 'urkud'] nobody
313-42767
10 months ago
501-35011
1 year ago
0-0
0 seconds
9146 laughinggas
author:laughinggas
feat(Data/ZMod/Defs): Topological structure on `ZMod` Added a discrete topology structure to `ZMod n` for all `n` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-topology merge-conflict awaiting-author
label:t-algebra$
55/3 Mathlib.lean,Mathlib/Topology/Algebra/Constructions.lean,Mathlib/Topology/Algebra/Group/Basic.lean,Mathlib/Topology/Instances/ZMod.lean,Mathlib/Topology/Maps.lean 5 61 ['YaelDillies', 'eric-wieser', 'github-actions', 'jcommelin', 'laughinggas', 'mo271', 'urkud'] nobody
313-42767
10 months ago
494-50895
1 year ago
7-6153
7 days
9229 eric-wieser
author:eric-wieser
refactor(Algebra/GradedMonoid): Use `HMul` to define `GMul` This make the notation much nicer, but I'm pretty sure this is a bad idea for performance / ambiguity reasons. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict WIP
label:t-algebra$
114/125 Mathlib/Algebra/DirectSum/Algebra.lean,Mathlib/Algebra/DirectSum/Internal.lean,Mathlib/Algebra/DirectSum/Ring.lean,Mathlib/Algebra/GradedMonoid.lean,Mathlib/Algebra/GradedMulAction.lean,Mathlib/Algebra/Module/GradedModule.lean,Mathlib/Algebra/MonoidAlgebra/ToDirectSum.lean,Mathlib/LinearAlgebra/TensorAlgebra/ToTensorPower.lean,Mathlib/LinearAlgebra/TensorPower.lean,Mathlib/LinearAlgebra/TensorProduct/Graded/Internal.lean,Mathlib/RingTheory/GradedAlgebra/Basic.lean 11 6 ['eric-wieser', 'leanprover-bot'] nobody
313-42767
10 months ago
477-32484
1 year ago
0-0
0 seconds
9354 chenyili0818
author:chenyili0818
feat: monotonicity of gradient on convex real-valued functions This file is based on Mathlib.Analysis.Calculus.Gradient.Basic, and describes the calculation properties co-authored-by: Ziyu Wang [tropicalfish910@gmail.com](mailto:tropicalfish910@gmail.com) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis merge-conflict awaiting-author 540/0 Mathlib.lean,Mathlib/Analysis/Convex/ConvexFunction.lean 2 15 ['github-actions', 'winstonyin'] nobody
313-42767
10 months ago
444-9456
1 year ago
22-72922
22 days
9356 alexjbest
author:alexjbest
feat: assumption? A little helper for replacing `assumption`s with `exact` statements quickly --- If this is approved I will add tests This begs the question of whether it might simply be better to add some sort of code action for "replace with trythis output" [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta merge-conflict awaiting-author 24/0 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Common.lean,Mathlib/Tactic/TryAssumption.lean 4 5 ['alexjbest', 'j-loreaux', 'jcommelin'] nobody
313-42767
10 months ago
496-63164
1 year ago
19-26304
19 days
8582 eric-wieser
author:eric-wieser
wip --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict 3/7 Mathlib/Algebra/Category/AlgebraCat/Monoidal.lean,Mathlib/LinearAlgebra/TensorProduct.lean 2 4 ['eric-wieser', 'leanprover-bot'] nobody
313-42767
10 months ago
564-29623
1 year ago
0-0
0 seconds
8658 eric-wieser
author:eric-wieser
feat: support right actions for `Con` This adds a new `Con.CompatibleSMul` typeclass that captures exactly the condition when `smul` descends to the quotient. I was not quite able to merge this with `MulAction.QuotientAction`: * The imports are such that the congruence relation `QuotientGroup.con` is not yet available in that file * `QuotientGroup.con` requires the subgroup to be normal, while `MulAction.QuotientAction` does not --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict awaiting-author
label:t-algebra$
80/18 Mathlib/GroupTheory/Congruence.lean,Mathlib/RingTheory/Congruence.lean 2 6 ['YaelDillies', 'eric-wieser'] nobody
313-42767
10 months ago
363-21421
11 months ago
29-65537
29 days
8503 thorimur
author:thorimur
feat: meta utils for `refine?` This PR introduces some metaprogramming infrastructure and utilities that are necessary for `refine?` (#8364). * `elabTermWithHoles'` (and `withCollectingNewGoalsFrom'`): a more configurable version of `elabTermWithHoles`, which allows: preserving the initial mvar type; *not* tagging untagged goals; and postponing mvars. * Some `Syntax` and `TSyntax` functionality, including: * `TSyntax.map`(`M`), for acting on `TSyntax` with functions `f : Syntax -> (m) Syntax` * Range operations: `includes` and `isEqByRange` * `setTrailingInfoBy?` and `unsetOriginalTrailing`, which is like `unsetTrailing`, but behaves as expected. * `Term.withoutModifyingState`, which does not allow unknown mvarIds to escape via the infotree * `hasNewErrors`, which runs a monad computation and returns the value along with `true` or `false` depending on whether new error messages have been logged * the option `pp.anonymousMVarSuffixes`, which can be set to `false` to replace all numeric suffixes of anonymous mvars with `✝`, which is useful in tandem with `#guard_msgs` for tests (but is essentially a workaround—although it can make some tactic states more legible). --- I'm open to suggestions on the location and name of the option/delaborator used for trimming the numeric suffixes of anonymous mvar names (which is used in the tests)—including whether or not it should exist in the first place, as it's essentially just a workaround. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta merge-conflict awaiting-author 312/5 Mathlib.lean,Mathlib/Lean/CoreM.lean,Mathlib/Lean/Elab/Tactic/ElabTerm.lean,Mathlib/Lean/Elab/Term.lean,Mathlib/Util/Delaborators.lean,Mathlib/Util/Syntax.lean 6 2 ['kmill', 'thorimur'] kmill
assignee:kmill
313-42767
10 months ago
515-53065
1 year ago
38-46649
38 days
9252 FR-vdash-bot
author:FR-vdash-bot
chore: remove redundant covariance instances, add priority I noticed that the following code is surprisingly slow. ``` lean import Mathlib count_heartbeats in example {n : ℕ} : CovariantClass (Fin (n + 1)) (Fin (n + 1)) (· + ·) (· < ·) := by try infer_instance sorry ``` This PR removed some redundant instances. The heartbeats have dropped from 19118 to 11450 (still too slow). Lean4 still seems to make some redundant attempts. See also https://github.com/leanprover-community/mathlib4/issues/6646#issuecomment-1691792488. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) slow-typeclass-synthesis t-order t-algebra merge-conflict awaiting-author WIP
label:t-algebra$
40/32 Mathlib/Algebra/CovariantAndContravariant.lean,Mathlib/Algebra/Order/Group/Defs.lean,Mathlib/Algebra/Order/Monoid/Defs.lean,Mathlib/CategoryTheory/Abelian/DiagramLemmas/Four.lean 4 8 ['FR-vdash-bot', 'leanprover-bot', 'urkud'] nobody
313-42767
10 months ago
371-86192
1 year ago
0-0
0 seconds
9339 FMLJohn
author:FMLJohn
feat (RingTheory/GradedAlgebra/HomogeneousIdeal): given a finitely generated homogeneous ideal of a graded semiring, construct a finite spanning set for the ideal which only contains homogeneous elements --- - [ ] depends on: #8187 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict
label:t-algebra$
402/4 Mathlib.lean,Mathlib/Algebra/DirectSum/Internal.lean,Mathlib/Algebra/GradedMonoid.lean,Mathlib/Algebra/Module/GradeZeroModule.lean,Mathlib/RingTheory/Finiteness.lean,Mathlib/RingTheory/GradedAlgebra/Basic.lean,Mathlib/RingTheory/GradedAlgebra/HomogeneousIdeal.lean,Mathlib/RingTheory/GradedAlgebra/Noetherian.lean 8 11 ['FMLJohn', 'github-actions', 'jjaassoonn', 'leanprover-community-mathlib4-bot'] nobody
313-42767
10 months ago
347-30684
11 months ago
0-0
0 seconds
9564 AntoineChambert-Loir
author:AntoineChambert-Loir
weaken commutativity assumptions for AdjoinRoot.lift and AdjoinRoot.liftHom I weaken a commutativity assumption for docs#AdjoinRoot.liftHom that the target algebra be commutative. It is only assumed to be a Semiring. For that, I need to generalize docs#AdjoinRoot.lift which takes `i : R ->+* S`, `a : S` with `f.eval₂ i a = 0` and defines `AdjoinRoot f ->+* S` that extends `i ` and sends `AdjoinRoot.root f` to `a`. --- The initial version of the PR was to define `AdjoinRoot.lift'` where `S` is only a Semiring, with the additional assumption `hcomm : ∀ r, Commute (i r) a` that the element `a` commutes with the image of `i`. @jcommelin suggested to provide this argument as an `autoParam`, filled in by an ad hoc `commutativity` tactic. However, such an argument cannot be made implicit and a first version required to have this argument given each time, most of the time by `_`, even for all subsequent lemmas, `AdjoinRoot.lift_mk`, etc. To avoid this, I tried to make this assumption a `⦃hcomm : ∀ r, Commute (i r) a⦄`. This appears to have some side effects that proofs using an `exact` tactic or in term mode do not work well, but one can resort on `by simp […]`. Maybe @eric-wieser or @Vierkantor will have opinions on that. In some cases one can still give the argument as `(hcomm := by commutativity)`. (There are 3 options : - separate lemmas for the fully commutative case and for the case where a proof is needed - using the `commutativity` tactic, but with an argument `_` sometimes - using the optional argument.) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict WIP
label:t-algebra$
146/30 Mathlib.lean,Mathlib/Algebra/Algebra/Basic.lean,Mathlib/Algebra/Algebra/Hom.lean,Mathlib/Algebra/Group/Commute/Defs.lean,Mathlib/RingTheory/AdjoinRoot.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Commutativity.lean,Mathlib/Tactic/Commutativity/Init.lean 8 14 ['AntoineChambert-Loir', 'Vierkantor', 'eric-wieser', 'jcommelin'] nobody
313-42767
10 months ago
335-23470
11 months ago
16-24540
16 days
9570 eric-wieser
author:eric-wieser
feat(Algebra/Star): Non-commutative generalization of `StarModule` [Zulip thread](https://leanprover.zulipchat.com/#narrow/stream/116395-maths/topic/Star.20modules.20over.20non-commutative.20scalars/near/383664005). Until we address #7152, we have to have both `StarModule` and `StarModule'`. To prove this generalization is useful, this shows that with it as an assumption, `TrivSqZeroExt` is a `StarRing`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra awaiting-CI merge-conflict WIP
label:t-algebra$
66/6 Mathlib/Algebra/Star/Basic.lean,Mathlib/Algebra/Star/Pi.lean,Mathlib/Algebra/Star/Prod.lean,Mathlib/Algebra/TrivSqZeroExt.lean 4 0 [] nobody
313-42767
10 months ago
406-32973
1 year ago
0-0
0 seconds
8585 thorimur
author:thorimur
chore: bench lean4#2944 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict 1/1 lean-toolchain 1 2 ['leanprover-bot', 'thorimur'] nobody
313-42767
10 months ago
564-47945
1 year ago*
0-0
0 seconds*
9487 eric-wieser
author:eric-wieser
feat: the exponential of dual numbers over non-commutative rings This is a work in progress, as I don't know my way around the measure theory library. --- - [x] depends on: #9489 - [x] depends on: #9486 - [x] depends on: #10427 - [ ] depends on: #10452 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-measure-probability t-algebra t-analysis merge-conflict WIP
label:t-algebra$
97/0 Mathlib/Analysis/NormedSpace/TrivSqZeroExt.lean 1 7 ['github-actions', 'leanprover-community-mathlib4-bot'] nobody
313-42767
10 months ago
318-37836
10 months ago
0-0
0 seconds
9504 alreadydone
author:alreadydone
chore: remove some IsSeparable assumptions --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict WIP
label:t-algebra$
41/14 Mathlib/NumberTheory/NumberField/Norm.lean,Mathlib/RingTheory/Norm.lean 2 0 [] nobody
313-42767
10 months ago
402-17551
1 year ago
0-0
0 seconds
9482 yuma-mizuno
author:yuma-mizuno
refactor(CategoryTheory/Monoidal): add `LaxMonoidalStruct` Add a `LaxMonoidalStruct` with only the unit morphism `ε` and the tensorator `μ`. This is used in #6307 to provide two different constructors for `LaxMonoidal` that have common `ε` and `μ` but use the tensor of morphisms or the whiskerings. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory merge-conflict WIP 21/8 Mathlib/Algebra/Category/ModuleCat/Adjunctions.lean,Mathlib/CategoryTheory/Monoidal/Functorial.lean,Mathlib/CategoryTheory/Monoidal/Limits.lean 3 0 [] nobody
313-42767
10 months ago
501-46616
1 year ago
0-0
0 seconds
9642 eric-wieser
author:eric-wieser
refactor(Analysis/Normed/{Group/Field}/Basic): Let `extends` generate the repeated fields New-style structure shenanigans mean that instance constructors randomly complain about a missing field that can be found with `__ : MetricSpace _ := infer_instance`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) I will write a longer PR description for this once CI is happy t-analysis merge-conflict awaiting-author WIP help-wanted 122/202 Mathlib/Analysis/Calculus/ContDiff/Basic.lean,Mathlib/Analysis/Complex/Basic.lean,Mathlib/Analysis/Matrix.lean,Mathlib/Analysis/Normed/Field/Basic.lean,Mathlib/Analysis/Normed/Group/Basic.lean,Mathlib/Analysis/Normed/Group/Completion.lean,Mathlib/Analysis/Normed/Order/Basic.lean,Mathlib/Analysis/NormedSpace/ProdLp.lean,Mathlib/Analysis/NormedSpace/Star/Matrix.lean,Mathlib/Analysis/NormedSpace/Unitization.lean,Mathlib/Analysis/Quaternion.lean,Mathlib/Geometry/Manifold/Instances/Sphere.lean,Mathlib/InformationTheory/Hamming.lean,Mathlib/MeasureTheory/Measure/Lebesgue/VolumeOfBalls.lean,Mathlib/NumberTheory/NumberField/CanonicalEmbedding.lean,Mathlib/NumberTheory/Padics/PadicIntegers.lean,Mathlib/Topology/ContinuousFunction/Bounded.lean 17 11 ['eric-wieser', 'leanprover-bot', 'urkud'] nobody
313-42767
10 months ago
491-22669
1 year ago
0-0
0 seconds
6630 MohanadAhmed
author:MohanadAhmed
feat: Reduced Spectral Theorem For A hermitian matrix $A : n \times n$ with rank $A.rank \leq n$, we can eliminate the zero eigenvalues and their corresponding eigenvectors from the (alternate) spectral theorem. As such the matrix $A$ can be written as: $$A = V₁ D V₁ᴴ$$ where - $V₁$ : $n \times r$ is the matrix of eigenvector with non-zero associated eigenvalues. - $D$ is $r \times r$ is the diagonal matrix containing only non-zero eigenvalues on its main diagonal. with $r = A.rank$ being the rank of the matrix Towards that goal we make several equivalence definitions: - `{i // hA.eigenvalues i ≠ 0} ≃ Fin (A.rank)` the set of non-zero eigenvalues can be indexed by the numbers from 0 to (r - 1). - `{i // ¬ hA.eigenvalues i ≠ 0} ≃ Fin (n - A.rank)` the set of non-zero eigenvalues can be indexed by the numbers from 0 to (n - r - 1). - `{i // hA.eigenvalues i ≠ 0} ⊕ {i // ¬hA.eigenvalues i ≠ 0} ≃ n`: the index set of the matrix (together with the associated eigenvector matrix and eigenvalues matrix ) can be partitioned into two complement groups the ones corresponding to non-zero eigenvalues and the ones corresponding to zero eigenvalues. - We can then put the previous definitions together to obtain a: `Fin (A.rank) ⊕ Fin (Fintype.card n - A.rank) ≃ n` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict WIP
label:t-algebra$
31/0 Mathlib/LinearAlgebra/Matrix/Spectrum.lean 1 0 [] nobody
313-42766
10 months ago
325-21483
10 months ago
0-0
0 seconds
8364 thorimur
author:thorimur
feat: `refine?` This PR adds `refine? e`, which suggests replacing unsynthesized `_`'s in `e` with `?_` in order to make `refine e'` work: ```lean example : Nat → Nat := by refine? fun (_ : _) => _ -- Try this: refine fun (_ : _) => ?_ ``` Note that this only suggests replacements for `_`'s present in the syntax; to create goals for implicit or instance arguments, the user is expected to use `refine'`. --- I'm especially open to suggestions on the filename (currently `RefineFix`). I'm also curious if this behaves as expected! Feel free to try it out "in real life" and comment here on edge cases. - [ ] depends on: #8503 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta merge-conflict blocked-by-other-PR 684/5 Mathlib.lean,Mathlib/Lean/CoreM.lean,Mathlib/Lean/Elab/Tactic/ElabTerm.lean,Mathlib/Lean/Elab/Term.lean,Mathlib/Tactic.lean,Mathlib/Tactic/RefineFix.lean,Mathlib/Util/Delaborators.lean,Mathlib/Util/Syntax.lean,test/RefineFix.lean 9 5 ['j-loreaux', 'leanprover-community-mathlib4-bot', 'thorimur'] nobody
313-42766
10 months ago
335-23470
11 months ago
6-59794
6 days
7351 shuxuezhuyi
author:shuxuezhuyi
feat(Topology/Algebra/Order): extend function on `Ioo` to `Icc` Extend a strictly monotone function defined on an open interval. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order merge-conflict awaiting-author 59/0 Mathlib.lean,Mathlib/Data/Set/Function.lean,Mathlib/Topology/Algebra/Order/IccExtendFromIoo.lean 3 7 ['j-loreaux', 'shuxuezhuyi'] nobody
313-42766
10 months ago
443-6032
1 year ago
30-30522
30 days
7227 kmill
author:kmill
feat: flexible binders and integration into notation3 Introduces `flexibleBinders`, which is an extensible system for binder notations that allow destructuring, bounded domains, and other niceties. Integrates this into `notation3`, and makes `Finset.sum`/`Finset.prod` use it. --- - [ ] depends on: #6833 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta merge-conflict WIP 1215/131 Mathlib.lean,Mathlib/Algebra/BigOperators/Basic.lean,Mathlib/Algebra/BigOperators/Intervals.lean,Mathlib/Algebra/BigOperators/NatAntidiagonal.lean,Mathlib/Mathport/Notation.lean,Mathlib/Util/FlexibleBinders.lean,Mathlib/Util/FlexibleBindersFinset.lean,Mathlib/Util/SyntaxFun.lean,test/FlexibleBinders.lean,test/notation3.lean 10 3 ['eric-wieser', 'kmill', 'leanprover-community-mathlib4-bot'] nobody
313-42766
10 months ago
516-24202
1 year ago
0-0
0 seconds
7909 mcdoll
author:mcdoll
fix(Tactic/Continuity): remove npowRec and add new tag for Continuous.pow --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology t-meta merge-conflict WIP 14/9 Mathlib/Tactic/Continuity.lean,Mathlib/Topology/Category/TopCat/Limits/Basic.lean,test/Continuity.lean 3 2 ['eric-wieser'] nobody
313-42766
10 months ago
588-69207
1 year ago
0-72515
20 hours
7225 jjaassoonn
author:jjaassoonn
some random stuff - Consider two commutative rings `R` and `S` and `X` and `(R, S)`-bimodule. Consider the tensor functor `(X ⊗[R] .)` from the category of `R`-modules to the category of `S`-modules and the hom functor `X →ₗ[S] .` from the category of `S`-modules to the category of `R`-modules, they form an adjunction. - direct limits of modules commute with tensor product - A proof of ![00HD](https://stacks.math.columbia.edu/tag/00HD) Three definitions for flatness: 1. in terms of injectiveness ```lean def Flat.injective : Prop := ∀ ⦃N N' : ModuleCat.{u} R⦄ (L : N ⟶ N'), Function.Injective L → Function.Injective ((tensorRight (ModuleCat.of R M)).map L) ``` 2. in terms of ideals ```lean def Flat.ideal : Prop := ∀ (I : Ideal R), Function.Injective (TensorProduct.lift ((lsmul R M).comp I.subtype)) ``` 3. in terms of finitely generated ideal ```lean def Flat.fg_ideal : Prop := ∀ ⦃I : Ideal R⦄ (_ : I.FG), Function.Injective (TensorProduct.lift ((lsmul R M).comp I.subtype)) ``` and they are all equivalent: ```lean lemma tfae : List.TFAE [ Flat.injective R M, Flat.ideal R M, Flat.fg_ideal R M ] := by ``` The dependencies between these changed files are: ``` Algebra.Module.LinearMap--------------------------------- | | | | v v Algebra.Category.ModuleCat.TensorProduct -----> Algebra.Character | | | v Algebra.DirectLimitAndTensorProduct -------------> RingTheory.Flat ``` to prove equivalence of other definitions, e.g. exact functor, tor, etc should be easier with this because the proof is will be categorical --- ------------- Some other stuff not about flatness 1. If $S$ is a submonoid and $I$ is maximally disjoint from $S$ then $I$ is prime 2. if $\mathfrak p$ is a minimal prime, then $x \in \mathfrak p$ implies that $x$ is a zero divisor 3. Noetherian rings has only finitely many minimal ideals 4. One version of [the prime avoidance lemma](https://en.wikipedia.org/wiki/Prime_avoidance_lemma): if $E$ is an addsubgroup of a ring and is mutiplicatively closed, and $\mathfrak p_i$ is some prime ideals, then not being any subset of the individual prime ideal implies that not being a subset of their union ---------- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict 1828/16 Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/TensorProduct.lean,Mathlib/Algebra/Character.lean,Mathlib/Algebra/DirectLimitAndTensorProduct.lean,Mathlib/Algebra/Module/LinearMap.lean,Mathlib/AlgebraicGeometry/PrimeSpectrum/Basic.lean,Mathlib/AlgebraicGeometry/PrimeSpectrum/Noetherian.lean,Mathlib/CategoryTheory/Functor/Fin.lean,Mathlib/CategoryTheory/ShortExactSequence.lean,Mathlib/RingTheory/Flat.lean,Mathlib/RingTheory/Ideal/Basic.lean,Mathlib/RingTheory/Ideal/MinimalPrime.lean,Mathlib/RingTheory/Ideal/PrimeAvoidance.lean 13 6 ['eric-wieser', 'jjaassoonn'] nobody
313-42766
10 months ago
507-21671
1 year ago
0-0
0 seconds
7875 FR-vdash-bot
author:FR-vdash-bot
chore: make `SMulCommClass A A B` and `SMulCommClass A B B` higher priority --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) slow-typeclass-synthesis t-algebra merge-conflict
label:t-algebra$
54/48 Mathlib/Algebra/Algebra/Basic.lean,Mathlib/Algebra/Algebra/NonUnitalSubalgebra.lean,Mathlib/Algebra/DirectSum/Algebra.lean,Mathlib/Algebra/Group/Action/Defs.lean,Mathlib/Algebra/Group/Subgroup/Actions.lean,Mathlib/Algebra/Lie/NonUnitalNonAssocAlgebra.lean,Mathlib/Algebra/Module/LinearMap/End.lean,Mathlib/Algebra/MonoidAlgebra/Basic.lean,Mathlib/Algebra/MvPolynomial/Basic.lean,Mathlib/Algebra/Ring/CentroidHom.lean,Mathlib/Algebra/Ring/Subring/Basic.lean,Mathlib/Algebra/Ring/Subsemiring/Basic.lean,Mathlib/Algebra/Star/NonUnitalSubalgebra.lean,Mathlib/Analysis/Complex/UnitDisc/Basic.lean,Mathlib/Analysis/NormedSpace/lpSpace.lean,Mathlib/Data/Matrix/Basic.lean,Mathlib/GroupTheory/GroupAction/Prod.lean,Mathlib/GroupTheory/GroupAction/Ring.lean,Mathlib/GroupTheory/GroupAction/SubMulAction.lean,Mathlib/GroupTheory/MonoidLocalization.lean,Mathlib/GroupTheory/Submonoid/Center.lean,Mathlib/LinearAlgebra/PiTensorProduct.lean,Mathlib/RingTheory/Ideal/Quotient.lean,Mathlib/RingTheory/TensorProduct/Basic.lean,Mathlib/Topology/ContinuousFunction/ContinuousMapZero.lean,Mathlib/Topology/ContinuousFunction/StoneWeierstrass.lean,Mathlib/Topology/ContinuousFunction/ZeroAtInfty.lean 27 15 ['FR-vdash-bot', 'Parcly-Taxel', 'jcommelin', 'leanprover-bot'] nobody
313-42766
10 months ago
335-23470
11 months ago
1-47913
1 day
6777 adomani
author:adomani
chore(Co*variantClass): replace eta-expanded (· * ·), (· + ·), (· ≤ ·), (· < ·) Replace `CovariantClass X X (· * ·) (· ≤ ·)` with -> `CovariantClass X X HMul.hMul LE.le` and similarly for `HAdd`, `LT`, `Contravariant`. This PR is inspired by [Issue #6646](https://github.com/leanprover-community/mathlib4/issues/6646) and, more specifically, [this comment](https://github.com/leanprover-community/mathlib4/issues/6646#issuecomment-1692792066). Note that https://github.com/leanprover/lean4/pull/2267 would make this unnecessary --- ```bash # First sed command: # the first captured pattern is `Co*variantClass ` # the second captured pattern is `` # the third captured pattern is `+` or `*` # the fourth captured pattern is `<` or `≤` # a match for `Co*variantClass ·) (· ·)` becomes # `Co*variantClass replaceop replaceop` # Second sed command: similar to the first, but looks for `(Function.swap (· ·))` sed -i ' s=\(Co[ntra]*variantClass \(..*\) \2 \)(· *\([+*]\) *·) (· *\([<≤]\) *·)=\1replaceop\3 replaceop\4=g s=\(Co[ntra]*variantClass \(..*\) \2 \)(\([Functio\.swap ]*\)(· *\([+*]\) *·)) (· *\([<≤]\) *·)=\1(\3replaceop\4) replaceop\5=g s=replaceop+=HAdd.hAdd=g s=replaceop\*=HMul.hMul=g s=replaceop<=LT.lt=g s=replaceop≤=LE.le=g s=\(Co[ntra]*variantClass N N\) (· \* ·) r=\1 HMul.hMul r=g s=\(Co[ntra]*variantClass N N (swap μ)\) (· ≤ ·)=\1 LE.le=g s=\(Co[ntra]*variantClass N N\) (swap (· \* ·)) r=\1 (swap HMul.hMul) r=g s=\(CovariantClass (Filter α) (Filter α)\) (· / ·) (· ≤ ·)=\1 HDiv.hDiv LE.le=g s=\(CovariantClass (Filter α) (Filter α)\) (swap (· / ·)) (· ≤ ·)=\1 (swap HDiv.hDiv) LE.le=g s=\(Co[ntra]*variantClass .* (fun x y .> . \* .)\) (· ≤ ·)=\1 LE.le=g s=\(Co[ntra]*variantClass .* (fun x y .> . \* .)\) (· < ·)=\1 LT.lt=g s=\(Co[ntra]*variantClass [^}]*\) (· ≤ ·)=\1 LE.le=g s=\(CovariantClass .* (Filter β)\) (· • ·) LE.le=\1 HSMul.hSMul LE.le=g ' $(git ls-files '*.lean') ``` [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict 703/678 Counterexamples/ZeroDivisorsInAddMonoidAlgebras.lean,Mathlib/Algebra/BigOperators/Basic.lean,Mathlib/Algebra/Bounds.lean,Mathlib/Algebra/CovariantAndContravariant.lean,Mathlib/Algebra/DirectSum/Internal.lean,Mathlib/Algebra/Group/UniqueProds.lean,Mathlib/Algebra/GroupPower/Order.lean,Mathlib/Algebra/MonoidAlgebra/Degree.lean,Mathlib/Algebra/Order/Archimedean.lean,Mathlib/Algebra/Order/Group/Abs.lean,Mathlib/Algebra/Order/Group/Defs.lean,Mathlib/Algebra/Order/Group/DenselyOrdered.lean,Mathlib/Algebra/Order/Group/MinMax.lean,Mathlib/Algebra/Order/Group/OrderIso.lean,Mathlib/Algebra/Order/Hom/Monoid.lean,Mathlib/Algebra/Order/Interval.lean,Mathlib/Algebra/Order/Kleene.lean,Mathlib/Algebra/Order/LatticeGroup.lean,Mathlib/Algebra/Order/Module.lean,Mathlib/Algebra/Order/Monoid/Basic.lean,Mathlib/Algebra/Order/Monoid/Cancel/Defs.lean,Mathlib/Algebra/Order/Monoid/Canonical/Defs.lean,Mathlib/Algebra/Order/Monoid/Defs.lean,Mathlib/Algebra/Order/Monoid/Lemmas.lean,Mathlib/Algebra/Order/Monoid/MinMax.lean,Mathlib/Algebra/Order/Monoid/NatCast.lean,Mathlib/Algebra/Order/Monoid/OrderDual.lean,Mathlib/Algebra/Order/Monoid/Prod.lean,Mathlib/Algebra/Order/Monoid/WithTop.lean,Mathlib/Algebra/Order/Monoid/WithZero/Basic.lean,Mathlib/Algebra/Order/Monoid/WithZero/Defs.lean,Mathlib/Algebra/Order/Nonneg/Ring.lean,Mathlib/Algebra/Order/Pointwise.lean,Mathlib/Algebra/Order/Positive/Ring.lean,Mathlib/Algebra/Order/Ring/Canonical.lean,Mathlib/Algebra/Order/Ring/Defs.lean,Mathlib/Algebra/Order/Ring/Lemmas.lean,Mathlib/Algebra/Order/Sub/Basic.lean,Mathlib/Algebra/Order/Sub/Canonical.lean,Mathlib/Algebra/Order/Sub/Defs.lean,Mathlib/Algebra/Order/WithZero.lean,Mathlib/Algebra/Parity.lean,Mathlib/Algebra/Star/Order.lean,Mathlib/Algebra/Tropical/Basic.lean,Mathlib/Analysis/Normed/Order/Lattice.lean,Mathlib/Data/DFinsupp/Lex.lean,Mathlib/Data/DFinsupp/Order.lean,Mathlib/Data/Finset/Fold.lean,Mathlib/Data/Finsupp/Lex.lean,Mathlib/Data/Finsupp/Order.lean,Mathlib/Data/List/BigOperators/Basic.lean,Mathlib/Data/List/BigOperators/Lemmas.lean,Mathlib/Data/Multiset/Basic.lean,Mathlib/Data/Nat/Cast/Order.lean,Mathlib/Data/PNat/Basic.lean,Mathlib/Data/Real/ENNReal.lean,Mathlib/Data/Real/NNReal.lean,Mathlib/Data/Set/Semiring.lean,Mathlib/Data/Sign.lean,Mathlib/MeasureTheory/Function/LpOrder.lean,Mathlib/MeasureTheory/Function/SimpleFuncDenseLp.lean,Mathlib/MeasureTheory/Measure/MeasureSpace.lean,Mathlib/MeasureTheory/Measure/VectorMeasure.lean,Mathlib/Order/ConditionallyCompleteLattice/Group.lean,Mathlib/Order/Filter/Basic.lean,Mathlib/Order/Filter/Pointwise.lean,Mathlib/Probability/Martingale/Basic.lean,Mathlib/Probability/Process/Stopping.lean,Mathlib/RingTheory/GradedAlgebra/Basic.lean,Mathlib/SetTheory/Cardinal/Basic.lean,Mathlib/SetTheory/Game/Basic.lean,Mathlib/SetTheory/Game/PGame.lean,Mathlib/SetTheory/Ordinal/Arithmetic.lean,Mathlib/SetTheory/Ordinal/Basic.lean,Mathlib/SetTheory/Ordinal/NaturalOps.lean,Mathlib/Tactic/GCongr/Core.lean,Mathlib/Tactic/Positivity/Basic.lean,Mathlib/Topology/ContinuousFunction/Algebra.lean,lean-toolchain,test/Recall.lean,test/propose.lean 81 36 ['adomani', 'alreadydone', 'digama0', 'eric-wieser', 'ericrbg', 'jcommelin', 'leanprover-bot', 'sgouezel'] nobody
313-42766
10 months ago
335-23470
11 months ago
35-56459
35 days
7615 eric-wieser
author:eric-wieser
chore(LinearAlgebra/Basic): generalize compatibleMaps to semilinear maps Spotted while reviewing #7611 --- - [x] depends on: #7611 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra awaiting-CI easy merge-conflict
label:t-algebra$
9/33 Mathlib/LinearAlgebra/Basic.lean 1 1 ['leanprover-community-mathlib4-bot'] nobody
313-42766
10 months ago
335-23470
11 months ago
0-0
0 seconds
7932 eric-wieser
author:eric-wieser
refactor(Algebra/TrivSqZeroExt): replace with a structure This is dogfooding my claim that "one-field structures are the lesser evil in Lean 4". This runs into the `simp [(stupid_parens)]` bug; or rather, a particular nasty instance of it where the offending simp call is inside `@[simps]`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra awaiting-CI merge-conflict
label:t-algebra$
155/73 Mathlib/Algebra/DualNumber.lean,Mathlib/Algebra/TrivSqZeroExt.lean,Mathlib/Logic/Equiv/TransferInstance.lean,Mathlib/Topology/Instances/TrivSqZeroExt.lean 4 1 ['github-actions'] nobody
313-42766
10 months ago
335-23470
11 months ago
0-0
0 seconds
7564 shuxuezhuyi
author:shuxuezhuyi
feat(Topology/Algebra/Order): extend strictly monotone function on `Ioo` to homeomorphism on `Icc` A strictly monotone function between open intervals can be extended to a homeomorphism between the closed intervals. --- - [ ] depends on: #7351 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology merge-conflict blocked-by-other-PR 162/0 Mathlib.lean,Mathlib/Topology/Algebra/Order/IccExtendFromIoo.lean 2 1 ['leanprover-community-mathlib4-bot'] nobody
313-42766
10 months ago
335-23470
11 months ago
0-0
0 seconds
7649 eric-wieser
author:eric-wieser
wip: instead of `suppress_compilation`, use `implemented_by` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP 7/14 Mathlib/LinearAlgebra/BilinearForm/TensorProduct.lean,Mathlib/LinearAlgebra/QuadraticForm/TensorProduct.lean,Mathlib/LinearAlgebra/TensorProduct.lean,Mathlib/LinearAlgebra/TensorProduct/Tower.lean,Mathlib/RingTheory/TensorProduct.lean 5 0 [] nobody
313-42766
10 months ago
455-49099
1 year ago
0-0
0 seconds
7427 MohanadAhmed
author:MohanadAhmed
Mohanad ahmed/sort eigenvalues abs In the file `Analysis.InnerProductSpace.Spectrum` todo notes were left saying: > TODO Postcompose with a permutation so that these eigenvectors are listed in increasing order of eigenvalue. > TODO Postcompose with a permutation so that these eigenvalues are listed in increasing order. - This is a start in that direction --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP 162/4 Mathlib/Analysis/InnerProductSpace/Spectrum.lean,Mathlib/Analysis/NormedSpace/PiLp.lean,Mathlib/LinearAlgebra/Matrix/Spectrum.lean 3 0 [] nobody
313-42766
10 months ago
490-69463
1 year ago
0-0
0 seconds
7835 shuxuezhuyi
author:shuxuezhuyi
feat(LinearAlgebra/Matrix): `lift` for projective special linear group We provide converters to help with the use of "quotient.liftOn" on projective special linear groups. --- - [x] depends on: #7826 - [x] depends on: #7791 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict awaiting-author
label:t-algebra$
52/0 Mathlib/LinearAlgebra/Matrix/ProjectiveSpecialLinearGroup.lean 1 3 ['jcommelin', 'leanprover-community-mathlib4-bot', 'shuxuezhuyi'] jcommelin
assignee:jcommelin
313-42766
10 months ago
333-82625
10 months ago
1-85757
1 day
7713 RemyDegenne
author:RemyDegenne
feat: add_left/right_inj for measures `μ + ν₁ = μ + ν₂ ↔ ν₁ = ν₂`, and similarly on the right. This is not true in general for measures, but is true when `μ` is mutually singular with the two other measures or when `μ` is finite. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-measure-probability merge-conflict awaiting-author 53/1 Mathlib/MeasureTheory/Measure/MutuallySingular.lean,lean-toolchain 2 6 ['RemyDegenne', 'digama0', 'eric-wieser', 'fpvandoorn'] nobody
313-42766
10 months ago
587-48606
1 year ago
0-62955
17 hours
6791 eric-wieser
author:eric-wieser
refactor: Use flat structures for morphisms This restores the symmetry we had in Lean3, where we had `MonoidHom.mk f one mul` not `MonoidHom.mk (OneHom.mk f one) mul`, and `f.toFun` wasn't notation for `f.toMulHom.toFun`. The nesting provided by the previous inheritance is useless to us in the face of `MonoidHomClass.toMonoidHom`, which completely eta-expands the structure anyway. We call the class `FunLikeFlatHack._` because this means the field is called `to_` which uses up less space in the goal view than any alternative. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-CI merge-conflict awaiting-author help-wanted 174/201 Mathlib/Algebra/Algebra/Equiv.lean,Mathlib/Algebra/Algebra/Hom.lean,Mathlib/Algebra/Category/GroupCat/ZModuleEquivalence.lean,Mathlib/Algebra/Category/GroupWithZeroCat.lean,Mathlib/Algebra/Category/ModuleCat/Presheaf.lean,Mathlib/Algebra/Category/MonCat/Basic.lean,Mathlib/Algebra/Group/Ext.lean,Mathlib/Algebra/Group/Prod.lean,Mathlib/Algebra/Group/UniqueProds.lean,Mathlib/Algebra/Hom/Equiv/Basic.lean,Mathlib/Algebra/Hom/Group/Defs.lean,Mathlib/Algebra/Hom/GroupAction.lean,Mathlib/Algebra/Hom/NonUnitalAlg.lean,Mathlib/Algebra/Hom/Ring/Defs.lean,Mathlib/Algebra/Lie/Basic.lean,Mathlib/Algebra/Module/Equiv.lean,Mathlib/Algebra/Module/LinearMap.lean,Mathlib/Algebra/Order/Hom/Ring.lean,Mathlib/Algebra/Order/Interval.lean,Mathlib/Algebra/Ring/Equiv.lean,Mathlib/Analysis/Normed/Group/SemiNormedGroupCat.lean,Mathlib/Data/FunLike/Basic.lean,Mathlib/Data/Rat/Cast/CharZero.lean,Mathlib/Data/Real/EReal.lean,Mathlib/Data/Real/Sqrt.lean,Mathlib/GroupTheory/FreeAbelianGroup.lean,Mathlib/GroupTheory/MonoidLocalization.lean,Mathlib/LinearAlgebra/Quotient.lean,Mathlib/LinearAlgebra/TensorProduct.lean,Mathlib/RingTheory/RingInvo.lean,Mathlib/Topology/Algebra/Module/Basic.lean,Mathlib/Topology/MetricSpace/Dilation.lean 32 0 [] nobody
313-42766
10 months ago
630-10626
1 year ago
0-0
0 seconds
7601 digama0
author:digama0
feat: ring hom support in `ring` As [requested on Zulip](https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/aroots/near/395750055). Adds support for distributing ring morphisms in `ring`: ```lean example (p : ℤ[X]) (r : ℤ) : C (2 * r) * p = C r * p + C r * p := by ring ``` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-meta merge-conflict awaiting-author
label:t-algebra$
257/48 Mathlib/Tactic/Ring/Basic.lean,test/linear_combination.lean,test/ring.lean 3 1 ['eric-wieser'] nobody
313-42766
10 months ago
370-53758
1 year ago
0-0
0 seconds
6930 kmill
author:kmill
feat: `resynth_instances` tactic for resynthesizing instances in the goal or local context This tactic can be useful for debugging non-canonical instances or for fixing up goals and hypotheses after using the `classical` tactic. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta merge-conflict WIP 327/0 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/ResynthInstances.lean,test/ResynthInstances.lean 4 0 [] nobody
313-42766
10 months ago
644-16789
1 year ago
0-0
0 seconds
6931 urkud
author:urkud
refactor(Analysis/Normed*): use `RingHomIsometric` for `*.norm_cast` --- I don't understand why linter fails. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis merge-conflict help-wanted 78/68 Mathlib/Analysis/LocallyConvex/ContinuousOfBounded.lean,Mathlib/Analysis/Normed/Field/Basic.lean,Mathlib/Analysis/Normed/Group/Basic.lean,Mathlib/Analysis/NormedSpace/Basic.lean,Mathlib/Analysis/NormedSpace/Exponential.lean,Mathlib/Analysis/NormedSpace/Spectrum.lean,Mathlib/Analysis/RCLike/Basic.lean,Mathlib/NumberTheory/NumberField/Embeddings.lean 8 0 [] nobody
313-42766
10 months ago
335-23470
11 months ago
0-0
0 seconds
6580 adomani
author:adomani
chore: `move_add`-driven replacements This PR accompanies #6576 and uses `move_add/mul` to simplify/streamline a selection of proofs. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author 12/13 Counterexamples/Monic_nonRegular.lean,Mathlib/Algebra/Associated.lean,Mathlib/Data/Polynomial/RingDivision.lean,Mathlib/LinearAlgebra/QuadraticForm/Basic.lean 4 0 [] nobody
313-42766
10 months ago
430-31198
1 year ago
0-0
0 seconds
7962 eric-wieser
author:eric-wieser
feat: `DualNumber (Quaternion R)` as a `CliffordAlgebra` This provides a clifford algebra isomorphic to the dual quaternions --- - [x] depends on: #7934 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict WIP
label:t-algebra$
307/7 Mathlib/Algebra/DualNumber.lean,Mathlib/Algebra/QuaternionBasis.lean,Mathlib/LinearAlgebra/CliffordAlgebra/Equivs.lean 3 16 ['github-actions', 'leanprover-community-mathlib4-bot'] nobody
313-42766
10 months ago
325-21355
10 months ago
0-0
0 seconds
7512 Komyyy
author:Komyyy
perf: override the data structures of coinductive types The data structures of the model of coinductive types (`Stream'`, `Computation`, `Stream'.Seq`) are inefficient, so we override their data structures. --- - [x] depends on: #7514 - [ ] depends on: leanprover/lean4#2292 - [x] depends on: leanprover/std4#371 - [x] depends on: #8460 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta merge-conflict blocked-by-core-PR blocked-by-other-PR WIP 6919/3700 Mathlib.lean,Mathlib/Algebra/ContinuedFractions/Basic.lean,Mathlib/Algebra/ContinuedFractions/Computation/ApproximationCorollaries.lean,Mathlib/Algebra/ContinuedFractions/Computation/Approximations.lean,Mathlib/Algebra/ContinuedFractions/Computation/Basic.lean,Mathlib/Algebra/ContinuedFractions/Computation/CorrectnessTerminating.lean,Mathlib/Algebra/ContinuedFractions/Computation/TerminatesIffRat.lean,Mathlib/Algebra/ContinuedFractions/Computation/Translations.lean,Mathlib/Algebra/ContinuedFractions/ContinuantRecurrence.lean,Mathlib/Algebra/ContinuedFractions/EvalEquiv.lean,Mathlib/Algebra/ContinuedFractions/Real.lean,Mathlib/Algebra/ContinuedFractions/TerminatedStable.lean,Mathlib/Algebra/ContinuedFractions/Translations.lean,Mathlib/Combinatorics/Hindman.lean,Mathlib/Control/Fix.lean,Mathlib/Control/LawfulFix.lean,Mathlib/Data/Seq/Computation.lean,Mathlib/Data/Seq/Parallel.lean,Mathlib/Data/Seq/Seq.lean,Mathlib/Data/Seq/WSeq.lean,Mathlib/Data/Stream.lean,lean-toolchain 22 2 ['digama0', 'leanprover-community-mathlib4-bot'] nobody
313-42766
10 months ago
375-20407
1 year ago
0-0
0 seconds
7467 ADedecker
author:ADedecker
feat: spectrum of X →ᵇ ℂ is StoneCech X --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis merge-conflict WIP 121/23 Mathlib/Analysis/NormedSpace/Star/BoundedContinuousFunction.lean,Mathlib/Analysis/NormedSpace/Star/GelfandDuality.lean,Mathlib/Topology/ContinuousFunction/Bounded.lean,Mathlib/Topology/ContinuousFunction/Compact.lean 4 1 ['github-actions'] nobody
313-42766
10 months ago
474-78178
1 year ago
0-0
0 seconds
4127 kmill
author:kmill
refactor: create HasAdj class, define Digraph, and generalize some SimpleGraph API --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics merge-conflict awaiting-author 1403/551 Mathlib.lean,Mathlib/Combinatorics/Digraph/Basic.lean,Mathlib/Combinatorics/Graph/Classes.lean,Mathlib/Combinatorics/Graph/Dart.lean,Mathlib/Combinatorics/Graph/Hom.lean,Mathlib/Combinatorics/SimpleGraph/AdjMatrix.lean,Mathlib/Combinatorics/SimpleGraph/Basic.lean,Mathlib/Combinatorics/SimpleGraph/Clique.lean,Mathlib/Combinatorics/SimpleGraph/Coloring.lean,Mathlib/Combinatorics/SimpleGraph/Connectivity.lean,Mathlib/Combinatorics/SimpleGraph/DegreeSum.lean,Mathlib/Combinatorics/SimpleGraph/Density.lean,Mathlib/Combinatorics/SimpleGraph/Ends/Defs.lean,Mathlib/Combinatorics/SimpleGraph/Finsubgraph.lean,Mathlib/Combinatorics/SimpleGraph/Hasse.lean,Mathlib/Combinatorics/SimpleGraph/Prod.lean,Mathlib/Combinatorics/SimpleGraph/StronglyRegular.lean,Mathlib/Combinatorics/SimpleGraph/Subgraph.lean 18 0 [] nobody
313-42765
10 months ago
354-40193
11 months ago
0-0
0 seconds
4785 thorimur
author:thorimur
feat: ExprWithLevels This introduces `ExprWithLevels`, a means of emulating universe polymorphism for non-constants during metaprogramming. [Description pending] - [ ] depends on: #4786 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta merge-conflict blocked-by-other-PR 491/1 Mathlib.lean,Mathlib/Lean/Meta/AppBuilder.lean,Mathlib/Lean/Meta/Basic.lean,Mathlib/Lean/Meta/ExprWithLevels.lean 4 1 ['kim-em'] nobody
313-42765
10 months ago
377-45989
1 year ago
0-0
0 seconds
6002 slerpyyy
author:slerpyyy
feat(Analysis.SpecialFunctions.Gaussian): add `integrable_fun_mul_exp_neg_mul_sq` If `f : ℝ → ℝ` is bounded by a polynomial, `fun x : ℝ => f x * exp (-b * x ^ 2)` is integrable. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis merge-conflict awaiting-author 26/0 Mathlib/Analysis/SpecialFunctions/Gaussian.lean 1 3 ['ocfnash', 'slerpyyy', 'urkud'] nobody
313-42765
10 months ago
578-32362
1 year ago
9-67365
9 days
6195 eric-wieser
author:eric-wieser
chore(RingTheory/TensorProduct): golf the `mul` definition --- - [x] depends on: #6211 - [x] depends on: #6187 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) Strangely this causes a timeout downstream t-algebra awaiting-CI merge-conflict
label:t-algebra$
4/29 Mathlib/RingTheory/TensorProduct.lean 1 1 ['leanprover-community-mathlib4-bot'] nobody
313-42765
10 months ago
335-23470
11 months ago
0-0
0 seconds
6590 mcdoll
author:mcdoll
feat: composition of LinearPMaps This PR changes the definition of the composition to allow composition of arbitrary LinearPMaps by restricting the domains appropriately. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict WIP
label:t-algebra$
51/7 Mathlib/LinearAlgebra/LinearPMap.lean,lean-toolchain 2 3 ['ADedecker', 'digama0', 'mcdoll'] nobody
313-42765
10 months ago
587-49372
1 year ago
3-26416
3 days
3575 Kha
author:Kha
perf: selectively enable precompilation --- This is an initial performance test on Linux. TODO: - [ ] test on macOS and Windows as well - [ ] adapt caching merge-conflict WIP 3/0 lakefile.lean 1 21 ['Kha', 'kim-em', 'leanprover-bot', 'tydeu'] nobody
313-42765
10 months ago
345-16360
11 months ago
0-0
0 seconds
4771 thorimur
author:thorimur
feat: Backtrack minimize Utilities for backtracking in order to attain a minimum according to some arbitrary notion of size when generating lists of parts and alternatives in alternating fashion. Motivated by minimizing the number of generated subgoals under apply-like actions on the goal. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta merge-conflict 482/1 Mathlib/Tactic/Backtracking.lean,test/Backtracking.lean 2 0 [] nobody
313-42765
10 months ago
635-62140
1 year ago
0-0
0 seconds
3808 kim-em
author:kim-em
feat: #formalize, backed by a choice of LLMs This replaces * https://github.com/leanprover-community/mathlib4/pull/3785, which has essentially been moved to an [independent repository](https://github.com/leanprover-community/llm) and generalised to interface with a choice of OpenAI's GPT, a gpt4all model (running locally via their python binding), or a model compatible with `llama.cpp` (e.g. the 4-bit quantised versions of Meta's LLaMa models). * https://github.com/leanprover-community/mathlib4/pull/3786, which has been modified slightly but still adds code here in `Mathlib.Tactic.Formalize`. Typical output: ``` #formalize "There are infinitely many primes numbers ending with a 7." ``` produces: * GPT4 ``` -- /-- There are infinitely many prime numbers ending with a 7. -/ -- theorem infinitely_many_primes_ending_with_7 : ∀ N : Nat, ∃ p, N < p ∧ p.Prime ∧ p % 10 = 7 := -- sorry ``` * ggml-gpt4all-j-v1.3-groovy.bin: ``` -- There are infinitely many prime numbers that end with a 7. ``` * 7B/ggml-model-q4_0.bin: ``` -- ∀ p : nat, 7 < 7p + 1 := sorry -– \end{code} ``` There are other sample outputs in `test/formalize.lean` If you don't currently have a LLM that the `leanprover-community/llm` project can recognise, when you run `#formalize` you get an error message, which currently reads: ``` Could not find a usable chat bot! You can try one of the following: * Obtain an OpenAI API access key at https://platform.openai.com/account/api-keys, and store it in the environment variable OPENAI_API_KEY. This will enable you to use ChatGPT. * Download the GPT4All-J model `https://gpt4all.io/models/ggml-gpt4all-j-v1.3-groovy.bin`, and put it in either `$HOME/.models/` or `$LLM_MODELS`. Also install the gpt4all python bindings via `pip3 install pygpt4all`. * Clone the `llama.cpp` repository from https://github.com/ggerganov/llama.cpp. Set the environment variable `LLAMA_CPP_HOME` to this repository. Follow the instructions in the README to produce `7B/ggml-model-q4_0.bin` starting from the Meta LLaMa weights. You can store this file at one of * `$LLAMA_CPP_HOME/models/7B/ggml-model-q4_0.bin` * `$HOME/.models/7B/ggml-model-q4_0.bin` * `$LLM_MODELS/7B/ggml-model-q4_0.bin` ``` Currently there are not user-configurable hooks to pick which LLM to use: it checks the conditions described in those bullet points, and takes the first one it finds. (i.e. if you want to use the LLaMa `7B/ggml-model-q4_0.bin`, you have to remove your OpenAI API key!). However a tactic in a downstream project (e.g. mathlib) can specify which interface and model it wants to use, or just call `findChatBot` for the behaviour described in that message. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta merge-conflict awaiting-author 180/0 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Formalize.lean,lake-manifest.json,lakefile.lean,test/formalize.lean 6 2 ['digama0', 'jcommelin'] nobody
313-42765
10 months ago
633-45893
1 year ago
124-45187
124 days
5133 kmill
author:kmill
feat: IntermediateField adjoin syntax for sets of elements Adds support for both `F⟮S⟯` and `F⟮α⟯`. The term `x` in `F⟮x⟯` is elaborated, and if it has type `Set _` the first interpretation is used, and otherwise the second is. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict WIP
label:t-algebra$
110/55 Mathlib/FieldTheory/Adjoin.lean 1 0 [] nobody
313-42765
10 months ago
668-81029
1 year ago
0-0
0 seconds
4775 thorimur
author:thorimur
feat: `SubExpr` utilities This file contains utilities for handling positions in expressions, including folding over subexpressions along with their positions. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta merge-conflict WIP 148/0 Mathlib.lean,Mathlib/Lean/SubExpr.lean 2 0 [] nobody
313-42765
10 months ago
733-54081
2 years ago
0-0
0 seconds
4109 kim-em
author:kim-em
feat: run library_search when the cursor is at a sorry --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta merge-conflict 77/0 Mathlib.lean,Mathlib/Data/Nondet/Basic.lean,Mathlib/Tactic/Common.lean,Mathlib/Tactic/LibrarySearch.lean,Mathlib/Util/CodeAction/RunTactic.lean 5 0 [] nobody
313-42765
10 months ago
521-62957
1 year ago
0-0
0 seconds
6403 FR-vdash-bot
author:FR-vdash-bot
chore: change instance priorities of `Ordered*` hierarchy --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) slow-typeclass-synthesis t-order t-algebra merge-conflict awaiting-author
label:t-algebra$
253/79 Mathlib/Algebra/Order/CompleteField.lean,Mathlib/Algebra/Order/Field/Canonical/Defs.lean,Mathlib/Algebra/Order/Field/Defs.lean,Mathlib/Algebra/Order/Group/Defs.lean,Mathlib/Algebra/Order/Monoid/Basic.lean,Mathlib/Algebra/Order/Monoid/Canonical/Defs.lean,Mathlib/Algebra/Order/Monoid/Defs.lean,Mathlib/Algebra/Order/Monoid/WithZero/Defs.lean,Mathlib/Algebra/Order/Ring/Canonical.lean,Mathlib/Algebra/Order/Ring/Defs.lean,Mathlib/Algebra/Order/Ring/Star.lean,Mathlib/Algebra/Order/WithZero.lean,Mathlib/Analysis/InnerProductSpace/Orientation.lean,Mathlib/LinearAlgebra/Orientation.lean,Mathlib/RingTheory/HahnSeries.lean,Mathlib/RingTheory/LaurentSeries.lean,Mathlib/Tactic/Positivity/Core.lean,Mathlib/Topology/Algebra/WithZeroTopology.lean 18 39 ['FR-vdash-bot', 'Vierkantor', 'digama0', 'eric-wieser', 'j-loreaux', 'leanprover-bot'] nobody
313-42765
10 months ago
371-86235
1 year ago
13-18399
13 days
7076 grunweg
author:grunweg
feat: define measure zero subsets of a manifold A topological manifold has no canonical measure, but there is a canonical notion of measure zero subsets. We show that these are closed under subsets and countable unions (hence define a filter, the almost everywhere filter) and that a closed nowhere dense has empty interior. This is necessary for stating the general version of Sard's theorem (in finite dimensions), and a first step towards its proof. This code was written at LftCM 2023. Thanks for @fpvandoorn for mentoring me! :heart: --- Unresolved questions/looking for feedback - Is "measure zero" a good name or would "null set" be better? I tend towards the former, but welcome input from a measure theorist (which I'm not). - What is the correct definition? One could also define "measure zero" using any `IsOpenPosMeasure` on the charted space. I think all results in this file still hold then, but for applications (e.g., Sard's theorem), this might be too general. - define custom notation, similar to the a.e. filter on a measure space? (We could include $J$ instead of $\mu$.) - what's the right syntax for formulas in docstrings --- use LaTeX or backticks? I don't know how to preview the generated docs, the guidelines are a bit ambiguous for me. t-measure-probability t-differential-geometry merge-conflict WIP 165/0 Mathlib.lean,Mathlib/Geometry/Manifold/MeasureZero.lean,docs/references.bib 3 27 ['ADedecker', 'github-actions', 'grunweg', 'mo271', 'sgouezel'] ADedecker
assignee:ADedecker
313-42765
10 months ago
352-38576
11 months ago
43-56043
43 days
6307 yuma-mizuno
author:yuma-mizuno
refactor(CategoryTheory/Monoidal): add whiskering operators We introduce whiskering operators. This allows us to introduce a simp-normal form for morphisms in monoidal categories. Rewriting into simp-normal forms is especially useful when combined with the coherence tactic. --- - [x] depends on: #6420 - [x] depends on: #8191 - [x] depends on: #9988 - [x] depends on: #9991 - [x] depends on: #9995 - [x] depends on: #10061 - [x] depends on: #10078 - [x] depends on: #10898 - [x] depends on: #10912 - [x] depends on: #11223 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory merge-conflict awaiting-author 325/280 Mathlib/Algebra/Category/ModuleCat/Adjunctions.lean,Mathlib/CategoryTheory/Bicategory/End.lean,Mathlib/CategoryTheory/Closed/Ideal.lean,Mathlib/CategoryTheory/Monoidal/Category.lean,Mathlib/CategoryTheory/Monoidal/Center.lean,Mathlib/CategoryTheory/Monoidal/Free/Basic.lean,Mathlib/CategoryTheory/Monoidal/Free/Coherence.lean,Mathlib/CategoryTheory/Monoidal/Functor.lean,Mathlib/CategoryTheory/Monoidal/FunctorCategory.lean,Mathlib/CategoryTheory/Monoidal/Limits.lean,Mathlib/CategoryTheory/Monoidal/Mon_.lean,Mathlib/CategoryTheory/Monoidal/NaturalTransformation.lean,Mathlib/CategoryTheory/Monoidal/Opposite.lean,Mathlib/CategoryTheory/Monoidal/Transport.lean,test/CategoryTheory/Coherence.lean 15 38 ['eric-wieser', 'github-actions', 'grunweg', 'jcommelin', 'kim-em', 'leanprover-community-mathlib4-bot', 'yuma-mizuno'] nobody
313-42765
10 months ago
328-55594
10 months ago
0-0
0 seconds
6633 adomani
author:adomani
feat(..Polynomial..): `MvPolynomial`s have no zero divisors This PR continues #6627, placing the `NoZeroDivisors` instance on `MvPolynomial`s and removing auxiliary intermediate results that are no longer needed. Affected files: ``` Data/MvPolynomial/Basic.lean Data/Polynomial/RingDivision.lean RingTheory/Polynomial/Basic.lean ``` --- - [ ] depends on: #6227 for the `NoZeroDivisors` instance on `AddMonoidAlgebra`s [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict awaiting-author
label:t-algebra$
143/57 Mathlib/Algebra/MonoidAlgebra/NoZeroDivisors.lean,Mathlib/Data/MvPolynomial/Basic.lean,Mathlib/Data/Polynomial/RingDivision.lean,Mathlib/RingTheory/Polynomial/Basic.lean 4 4 ['adomani', 'eric-wieser', 'leanprover-community-mathlib4-bot'] nobody
313-42765
10 months ago
660-4290
1 year ago
0-19160
5 hours
6330 FR-vdash-bot
author:FR-vdash-bot
chore: make some instance about `Sub...Class` higher priority than `Sub...` The opposite direction to #6328. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) slow-typeclass-synthesis t-algebra merge-conflict WIP
label:t-algebra$
123/128 Mathlib/Algebra/Algebra/NonUnitalSubalgebra.lean,Mathlib/Algebra/Algebra/Subalgebra/Basic.lean,Mathlib/Algebra/Star/NonUnitalSubalgebra.lean,Mathlib/FieldTheory/IsAlgClosed/Basic.lean,Mathlib/FieldTheory/Subfield.lean,Mathlib/RingTheory/NonUnitalSubring/Basic.lean,Mathlib/RingTheory/NonUnitalSubsemiring/Basic.lean,Mathlib/RingTheory/Polynomial/Quotient.lean,Mathlib/RingTheory/Subring/Basic.lean,Mathlib/RingTheory/Subsemiring/Basic.lean,lean-toolchain 11 13 ['FR-vdash-bot', 'digama0', 'leanprover-bot'] nobody
313-42765
10 months ago
371-86255
1 year ago
0-0
0 seconds
6993 jjaassoonn
author:jjaassoonn
feat : lemmas about `AddMonoidAlgebra.{divOf, modOf}` --- - [x] depends on: #7582 - [x] depends on: #8975 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict
label:t-algebra$
147/3 Mathlib/Algebra/MonoidAlgebra/Division.lean,Mathlib/Data/Finsupp/Basic.lean,Mathlib/Data/MvPolynomial/Basic.lean,Mathlib/Data/MvPolynomial/CommRing.lean,Mathlib/Data/MvPolynomial/Division.lean 5 42 ['YaelDillies', 'alreadydone', 'digama0', 'eric-wieser', 'github-actions', 'jjaassoonn', 'leanprover-community-mathlib4-bot'] nobody
313-42765
10 months ago
335-23470
11 months ago
102-21189
102 days
6491 eric-wieser
author:eric-wieser
chore(Mathlib/Algebra/Hom/GroupAction): add `SMulHomClass.comp_smul` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict
label:t-algebra$
24/10 Mathlib/Algebra/Hom/GroupAction.lean 1 0 [] nobody
313-42765
10 months ago
335-23470
11 months ago
83-76369
83 days
5912 ADedecker
author:ADedecker
feat(Analysis.Distribution.ContDiffMapSupportedIn): space of smooth maps with support in a fixed compact --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis merge-conflict WIP 513/13 Mathlib.lean,Mathlib/Analysis/Distribution/ContDiffMapSupportedIn.lean,Mathlib/Analysis/LocallyConvex/WithSeminorms.lean,Mathlib/Analysis/Seminorm.lean,Mathlib/Data/FunLike/Basic.lean,Mathlib/Data/Set/Function.lean,Mathlib/Topology/Algebra/Module/StrongTopology.lean,Mathlib/Topology/ContinuousFunction/Bounded.lean 8 0 [] nobody
313-42765
10 months ago
664-10406
1 year ago
0-0
0 seconds
6210 MohanadAhmed
author:MohanadAhmed
feat(Data/IsROrC/Basic): add a `StarOrderedRing` instance This PR implements a suggestion by @urkud on [Zulip thread](https://leanprover.zulipchat.com/#narrow/stream/113488-general/topic/PartialOrder.20and.20StarOrderedRing.20on.20IsROrC) on how to get a `StarOrderedRing` on the `IsROrC` class. In that discussion the suggested step were: 1. Add PartialOrder K to the list of extends and add le_iff_re_im : z ≤ w ↔ re z ≤ re w ∧ im z = im w to the list of axioms. 2. Prove StarOrderedRing instance for any IsROrC. 3. Add (almost trivial) le_iff_re_im proofs to IsROrC instances for real and complex numbers. This PR does exactly these three steps --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-analysis merge-conflict WIP
label:t-algebra$
25/24 Mathlib/Analysis/Complex/Basic.lean,Mathlib/Analysis/SpecialFunctions/Pow/Deriv.lean,Mathlib/Data/Complex/Basic.lean,Mathlib/Data/IsROrC/Basic.lean 4 19 ['MohanadAhmed', 'eric-wieser', 'j-loreaux'] nobody
313-42765
10 months ago
664-45902
1 year ago
0-4269
1 hour
6328 FR-vdash-bot
author:FR-vdash-bot
chore: make some instance about `Sub...Class` lower priority Many similar instances have been marked as lower priority. I'd like to see if this would make things faster. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra awaiting-CI merge-conflict WIP
label:t-algebra$
14/14 Mathlib/RingTheory/NonUnitalSubsemiring/Basic.lean,Mathlib/RingTheory/Subsemiring/Basic.lean,lean-toolchain 3 1 ['digama0'] nobody
313-42765
10 months ago
587-49373
1 year ago
0-0
0 seconds
6268 eric-wieser
author:eric-wieser
Fixups to #3838 This is an attempt to make #3838 universe polymorphic --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) * Depends on #6271 * Depends on #8876 merge-conflict WIP 186/107 Mathlib/Control/Random.lean,Mathlib/Tactic/SlimCheck.lean,Mathlib/Testing/SlimCheck/Functions.lean,Mathlib/Testing/SlimCheck/Gen.lean,Mathlib/Testing/SlimCheck/Sampleable.lean,Mathlib/Testing/SlimCheck/Testable.lean,test/slim_check.lean 7 10 ['github-actions', 'kim-em'] nobody
313-42765
10 months ago
539-74632
1 year ago
0-0
0 seconds
5934 eric-wieser
author:eric-wieser
feat: port Data.Rat.MetaDefs --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) This needs some eyes from people familiar with Qq t-meta merge-conflict mathlib-port help-wanted 183/0 Mathlib.lean,Mathlib/Data/Rat/MetaDefs.lean,test/rat.lean 3 4 ['eric-wieser', 'gebner'] nobody
313-42765
10 months ago
483-29754
1 year ago
0-0
0 seconds
4960 eric-wieser
author:eric-wieser
chore: use `open scoped` Earlier versions of mathport did not know about this. This was done by searching for all `open` commands referencing: * `Classical` * `BigOperators` * `Topology` * `Pointwise` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-CI merge-conflict 1026/981 Mathlib/Algebra/AddTorsor.lean,Mathlib/Algebra/Algebra/Basic.lean,Mathlib/Algebra/Algebra/Equiv.lean,Mathlib/Algebra/Algebra/Hom.lean,Mathlib/Algebra/Algebra/Operations.lean,Mathlib/Algebra/Algebra/Subalgebra/Basic.lean,Mathlib/Algebra/Algebra/Subalgebra/Pointwise.lean,Mathlib/Algebra/Algebra/Subalgebra/Tower.lean,Mathlib/Algebra/Algebra/Tower.lean,Mathlib/Algebra/BigOperators/Associated.lean,Mathlib/Algebra/BigOperators/Basic.lean,Mathlib/Algebra/BigOperators/Fin.lean,Mathlib/Algebra/BigOperators/Finprod.lean,Mathlib/Algebra/BigOperators/Finsupp.lean,Mathlib/Algebra/BigOperators/Intervals.lean,Mathlib/Algebra/BigOperators/NatAntidiagonal.lean,Mathlib/Algebra/BigOperators/Option.lean,Mathlib/Algebra/BigOperators/Order.lean,Mathlib/Algebra/BigOperators/Pi.lean,Mathlib/Algebra/BigOperators/Ring.lean,Mathlib/Algebra/BigOperators/RingEquiv.lean,Mathlib/Algebra/Bounds.lean,Mathlib/Algebra/Category/GroupCat/Biproducts.lean,Mathlib/Algebra/Category/GroupCat/FilteredColimits.lean,Mathlib/Algebra/Category/GroupCat/Injective.lean,Mathlib/Algebra/Category/ModuleCat/Adjunctions.lean,Mathlib/Algebra/Category/ModuleCat/Biproducts.lean,Mathlib/Algebra/Category/Mon/FilteredColimits.lean,Mathlib/Algebra/Category/Ring/Adjunctions.lean,Mathlib/Algebra/Category/Ring/FilteredColimits.lean,Mathlib/Algebra/CharP/Basic.lean,Mathlib/Algebra/CharP/Two.lean,Mathlib/Algebra/DirectLimit.lean,Mathlib/Algebra/DirectSum/Basic.lean,Mathlib/Algebra/DirectSum/Decomposition.lean,Mathlib/Algebra/DirectSum/Internal.lean,Mathlib/Algebra/DirectSum/Ring.lean,Mathlib/Algebra/EuclideanDomain/Defs.lean,Mathlib/Algebra/Field/Defs.lean,Mathlib/Algebra/GCDMonoid/Div.lean,Mathlib/Algebra/GeomSum.lean,Mathlib/Algebra/GroupWithZero/Basic.lean,Mathlib/Algebra/GroupWithZero/Commute.lean,Mathlib/Algebra/GroupWithZero/Units/Basic.lean,Mathlib/Algebra/Homology/Additive.lean,Mathlib/Algebra/Homology/ComplexShape.lean,Mathlib/Algebra/Homology/Homology.lean,Mathlib/Algebra/Homology/Homotopy.lean,Mathlib/Algebra/Homology/HomotopyCategory.lean,Mathlib/Algebra/Homology/ImageToKernel.lean,Mathlib/Algebra/IndicatorFunction.lean,Mathlib/Algebra/LinearRecurrence.lean,Mathlib/Algebra/Module/BigOperators.lean,Mathlib/Algebra/Module/GradedModule.lean,Mathlib/Algebra/Module/LinearMap.lean,Mathlib/Algebra/Module/PointwisePi.lean,Mathlib/Algebra/Module/Submodule/Basic.lean,Mathlib/Algebra/Module/Submodule/Bilinear.lean,Mathlib/Algebra/Module/Submodule/Lattice.lean,Mathlib/Algebra/Module/Submodule/Pointwise.lean,Mathlib/Algebra/Module/Torsion.lean,Mathlib/Algebra/MonoidAlgebra/Basic.lean,Mathlib/Algebra/MonoidAlgebra/Degree.lean,Mathlib/Algebra/Order/Chebyshev.lean,Mathlib/Algebra/Order/Module.lean,Mathlib/Algebra/Order/Pointwise.lean,Mathlib/Algebra/Order/Rearrangement.lean,Mathlib/Algebra/Order/SMul.lean,Mathlib/Algebra/Order/UpperLower.lean,Mathlib/Algebra/Periodic.lean,Mathlib/Algebra/Polynomial/BigOperators.lean,Mathlib/Algebra/Polynomial/GroupRingAction.lean,Mathlib/Algebra/Star/BigOperators.lean,Mathlib/Algebra/Star/Pointwise.lean,Mathlib/Algebra/Star/Subalgebra.lean,Mathlib/Algebra/Support.lean,Mathlib/Algebra/TrivSqZeroExt.lean,Mathlib/Algebra/Tropical/BigOperators.lean,Mathlib/AlgebraicGeometry/PrimeSpectrum/Basic.lean,Mathlib/AlgebraicGeometry/PrimeSpectrum/Maximal.lean,Mathlib/AlgebraicGeometry/ProjectiveSpectrum/Topology.lean,Mathlib/AlgebraicTopology/AlternatingFaceMapComplex.lean,Mathlib/AlgebraicTopology/ExtraDegeneracy.lean,Mathlib/AlgebraicTopology/TopologicalSimplex.lean,Mathlib/Analysis/Analytic/Basic.lean,Mathlib/Analysis/Asymptotics/AsymptoticEquivalent.lean,Mathlib/Analysis/Asymptotics/Asymptotics.lean,Mathlib/Analysis/Asymptotics/SpecificAsymptotics.lean,Mathlib/Analysis/Asymptotics/SuperpolynomialDecay.lean,Mathlib/Analysis/Asymptotics/Theta.lean,Mathlib/Analysis/BoxIntegral/Box/Basic.lean,Mathlib/Analysis/BoxIntegral/Box/SubboxInduction.lean,Mathlib/Analysis/BoxIntegral/Partition/Additive.lean,Mathlib/Analysis/BoxIntegral/Partition/Basic.lean,Mathlib/Analysis/BoxIntegral/Partition/Filter.lean,Mathlib/Analysis/BoxIntegral/Partition/Split.lean,Mathlib/Analysis/BoxIntegral/Partition/SubboxInduction.lean,Mathlib/Analysis/BoxIntegral/Partition/Tagged.lean,Mathlib/Analysis/Calculus/ContDiffDef.lean,Mathlib/Analysis/Calculus/Deriv/Add.lean 788 0 [] nobody
313-42765
10 months ago
335-23470
11 months ago
0-0
0 seconds
6079 eric-wieser
author:eric-wieser
fix: deduplicate variables `variables {A} [Ring A]` meant "update the binder of `A`" in Lean 3, but now means "create a duplicate variable called `A`" (or at least, does so when inspecting the state within the variables line). This removes a number of porting notes that were stumbling over this behavior. [Related Zulip thread](https://leanprover.zulipchat.com/#narrow/stream/270676-lean4/topic/unexpected.20.60variable.60.20behaviour.3F/near/360154080) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-CI merge-conflict 1012/443 Archive/Wiedijk100Theorems/CubingACube.lean,Mathlib/Algebra/Category/ModuleCat/Adjunctions.lean,Mathlib/Algebra/CharP/Basic.lean,Mathlib/Algebra/CovariantAndContravariant.lean,Mathlib/Algebra/DirectLimit.lean,Mathlib/Algebra/DirectSum/Finsupp.lean,Mathlib/Algebra/DirectSum/Module.lean,Mathlib/Algebra/GradedMonoid.lean,Mathlib/Algebra/Group/Pi.lean,Mathlib/Algebra/GroupPower/Basic.lean,Mathlib/Algebra/GroupPower/Lemmas.lean,Mathlib/Algebra/Hom/Aut.lean,Mathlib/Algebra/Hom/Equiv/Basic.lean,Mathlib/Algebra/Hom/Group.lean,Mathlib/Algebra/Homology/HomologicalComplex.lean,Mathlib/Algebra/Homology/HomotopyCategory.lean,Mathlib/Algebra/Homology/ImageToKernel.lean,Mathlib/Algebra/Homology/ShortComplex/LeftHomology.lean,Mathlib/Algebra/IndicatorFunction.lean,Mathlib/Algebra/Jordan/Basic.lean,Mathlib/Algebra/Lie/Classical.lean,Mathlib/Algebra/Lie/Subalgebra.lean,Mathlib/Algebra/Lie/Submodule.lean,Mathlib/Algebra/Lie/TensorProduct.lean,Mathlib/Algebra/Module/Injective.lean,Mathlib/Algebra/Module/LinearMap.lean,Mathlib/Algebra/Module/Submodule/Basic.lean,Mathlib/Algebra/MonoidAlgebra/Basic.lean,Mathlib/Algebra/MonoidAlgebra/Grading.lean,Mathlib/Algebra/Order/CompleteField.lean,Mathlib/Algebra/Order/Pi.lean,Mathlib/Algebra/Order/Ring/Lemmas.lean,Mathlib/Algebra/Ring/Equiv.lean,Mathlib/Algebra/SMulWithZero.lean,Mathlib/Algebra/Star/Module.lean,Mathlib/Algebra/Support.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Point.lean,Mathlib/AlgebraicGeometry/Morphisms/RingHomProperties.lean,Mathlib/AlgebraicGeometry/ProjectiveSpectrum/Scheme.lean,Mathlib/AlgebraicGeometry/StructureSheaf.lean,Mathlib/AlgebraicTopology/DoldKan/Decomposition.lean,Mathlib/AlgebraicTopology/MooreComplex.lean,Mathlib/Analysis/Calculus/ContDiff.lean,Mathlib/Analysis/Calculus/FormalMultilinearSeries.lean,Mathlib/Analysis/Calculus/LocalExtr.lean,Mathlib/Analysis/Calculus/TangentCone.lean,Mathlib/Analysis/Convex/Basic.lean,Mathlib/Analysis/Convex/Combination.lean,Mathlib/Analysis/Convex/Extreme.lean,Mathlib/Analysis/Convex/Function.lean,Mathlib/Analysis/Convex/Hull.lean,Mathlib/Analysis/Convex/Independent.lean,Mathlib/Analysis/Convex/Intrinsic.lean,Mathlib/Analysis/Convex/Join.lean,Mathlib/Analysis/Convex/Quasiconvex.lean,Mathlib/Analysis/Convex/Segment.lean,Mathlib/Analysis/Convex/Star.lean,Mathlib/Analysis/Convex/Uniform.lean,Mathlib/Analysis/Convolution.lean,Mathlib/Analysis/Fourier/RiemannLebesgueLemma.lean,Mathlib/Analysis/InnerProductSpace/Calculus.lean,Mathlib/Analysis/LocallyConvex/AbsConvex.lean,Mathlib/Analysis/LocallyConvex/BalancedCoreHull.lean,Mathlib/Analysis/LocallyConvex/Basic.lean,Mathlib/Analysis/LocallyConvex/Bounded.lean,Mathlib/Analysis/LocallyConvex/WithSeminorms.lean,Mathlib/Analysis/Normed/Field/Basic.lean,Mathlib/Analysis/Normed/Group/AddCircle.lean,Mathlib/Analysis/Normed/Group/Hom.lean,Mathlib/Analysis/Normed/Group/Seminorm.lean,Mathlib/Analysis/NormedSpace/Completion.lean,Mathlib/Analysis/NormedSpace/LinearIsometry.lean,Mathlib/Analysis/NormedSpace/Multilinear.lean,Mathlib/Analysis/NormedSpace/OperatorNorm.lean,Mathlib/Analysis/ODE/PicardLindelof.lean,Mathlib/Analysis/Seminorm.lean,Mathlib/CategoryTheory/Action.lean,Mathlib/CategoryTheory/Bicategory/LocallyDiscrete.lean,Mathlib/CategoryTheory/Bicategory/NaturalTransformation.lean,Mathlib/CategoryTheory/Closed/Ideal.lean,Mathlib/CategoryTheory/ConcreteCategory/UnbundledHom.lean,Mathlib/CategoryTheory/Core.lean,Mathlib/CategoryTheory/Endofunctor/Algebra.lean,Mathlib/CategoryTheory/Enriched/Basic.lean,Mathlib/CategoryTheory/EssentialImage.lean,Mathlib/CategoryTheory/FullSubcategory.lean,Mathlib/CategoryTheory/Functor/Category.lean,Mathlib/CategoryTheory/Limits/Fubini.lean,Mathlib/CategoryTheory/Limits/HasLimits.lean,Mathlib/CategoryTheory/Limits/Preserves/Shapes/Kernels.lean,Mathlib/CategoryTheory/Limits/Shapes/BinaryProducts.lean,Mathlib/CategoryTheory/Limits/Shapes/Biproducts.lean,Mathlib/CategoryTheory/Limits/Shapes/Equalizers.lean,Mathlib/CategoryTheory/Limits/Shapes/Images.lean,Mathlib/CategoryTheory/Limits/Shapes/WidePullbacks.lean,Mathlib/CategoryTheory/Linear/LinearFunctor.lean,Mathlib/CategoryTheory/Localization/Construction.lean,Mathlib/CategoryTheory/Monoidal/Braided.lean,Mathlib/CategoryTheory/Monoidal/CommMon_.lean,Mathlib/CategoryTheory/Monoidal/Discrete.lean 302 1 ['timotree3'] nobody
313-42765
10 months ago
335-23470
11 months ago
0-0
0 seconds
4871 j-loreaux
author:j-loreaux
feat: define the additive submonoid of positive elements in a star ordered ring This file defines the `AddSubmonoid` of nonegative elements `StarOrderedRing.positive R` in a star ordered ring `R` with carrier `{ x : R | 0 ≤ x }` (in fact, the definition only requires `OrderedAddCommMonoid R` to allow for other use cases, but it is primarily intended for `StarOrderedRing R`). Equivalently, this is the `AddSubmonoid` generated by the elements of the form `star s * s`. Even though this technically corresponds to the nonnegative elements, the "positive" terminology is standard throughout the literature (at least in C⋆-algebra theory and operator theory), so we choose to prefer that. The advantage of using this over other definitions of positivity is that it allows us to unify several different concepts under a single umbrella. For example, one might be tempted to consider the collection of bounded linear operators on an Hilbert space and define positivity as `∀ x, 0 ≤ ⟪T x, x⟫`, but this doesn't generalize nicely to C⋆-algebras. Alternatively, one could define positivity as those self-adjoint elements with nonnegative spectrum, but this requires the algebra to be unital. Our definition herein conveniently sidesteps these issues. --- Note: I declared the `AddMonoidWithOne` and `AddGroupWithOne` instances for `selfAdjoint R` separately because it made the proof of the latter easier. - [x] depends on: #6229 - [x] depends on: #10209 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra awaiting-CI merge-conflict
label:t-algebra$
216/12 Mathlib.lean,Mathlib/Algebra/Order/Ring/CharZero.lean,Mathlib/Algebra/Star/Order.lean,Mathlib/Algebra/Star/Positive.lean,Mathlib/Algebra/Star/SelfAdjoint.lean,Mathlib/GroupTheory/Submonoid/Operations.lean 6 28 ['eric-wieser', 'j-loreaux', 'leanprover-community-mathlib4-bot'] nobody
313-42765
10 months ago
335-23470
11 months ago
5-55287
5 days
3757 thorimur
author:thorimur
feat: config options for `fail_if_no_progress` This PR creates config options for `fail_if_no_progress` that allow the user to tweak what exactly counts as "progress". This includes whether to use defeq or `BEq`, what transparency to use, and which parts of the goal and local context to check. It also splits off the comparison functionality into `Mathlib.Lean.Meta.Compare`, which provides fully configurable comparison functions for common complex metaprogramming types not specific to `fail_if_no_progress`. These types are `Expr`, `LocalDecl`, `LocalContext`, `MetavarDecl`, `MVarId`, and `List MVarId`. --- See [zulip](https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/progress.20on.20fail_if_no_progress) for a couple review questions. Status update: this PR is now basically done, save for some extra tests which should probably be included. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta merge-conflict WIP 603/54 Mathlib.lean,Mathlib/Lean/Meta.lean,Mathlib/Lean/Meta/Compare.lean,Mathlib/Tactic/FailIfNoProgress.lean,test/fail_if_no_progress.lean 5 38 ['alexjbest', 'github-actions', 'joneugster', 'kim-em', 'thorimur'] nobody
313-42764
10 months ago
565-53950
1 year ago
45-49113
45 days
12353 thorimur
author:thorimur
feat: `conv%` This PR introduces `conv% e => tac`, along with `simp%`, `norm_num%`, and `push_neg%`, which are defined in terms of `conv%`. It also introduces `conv%?` (and `simp%?`, `norm_num%?`, and `push_neg%?`) as shortcuts for `show_term ...`. This is a relatively straightforward refactor of code already present in the implementation of `#conv`, and otherwise relies entirely on simple macros. This PR also introduces some modifications to existing command syntax for `#conv`, `#simp`, and `#norm_num`: * The syntax for `#conv` was `#conv tac => e`; however, this is inconsistent with the tactic syntax, and so this has been flipped to `#conv e => tac`. Likewise, `conv%` uses the same (new) syntax `conv% e => tac`. * `#simp` and `#norm_num` separated their config and `only` syntax from the expression by an optional `=>` (for `#simp`) and an optional `:` (for `#norm_num`) (e.g. `#simp only [lem] => e`). These have both been replaced with an optional`on` (e.g. `#simp only [lem] on e`) which is also used for `simp%` and `norm_num%`. Although `#whnf` is implemented in terms of `#conv`, this PR doesn't introduce `whnf%` in the same way, as that's probably better off being implemented directly instead of through `conv`. --- WIP: needs tests. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta merge-conflict WIP 131/32 Mathlib/Tactic/Conv.lean,Mathlib/Tactic/NormNum/Core.lean,Mathlib/Tactic/PushNeg.lean,docs/Conv/Guide.lean 4 0 [] nobody
309-19074
10 months ago
309-19074
10 months ago
0-0
0 seconds
13852 FR-vdash-bot
author:FR-vdash-bot
perf: skip some typeclasses in TC search --- - [ ] depends on: #7873 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) slow-typeclass-synthesis merge-conflict blocked-by-other-PR 45/33 Mathlib/Algebra/Group/Defs.lean,Mathlib/Algebra/Ring/Defs.lean,Mathlib/RingTheory/Norm.lean 3 21 ['FR-vdash-bot', 'MichaelStollBayreuth', 'github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot'] nobody
309-12754
10 months ago
309-12755
10 months ago
0-0
0 seconds
7903 urkud
author:urkud
feat: define `UnboundedSpace` --- The new instances generate some timeouts, and I don't understand why. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology merge-conflict help-wanted 111/59 Mathlib/Analysis/BoxIntegral/Basic.lean,Mathlib/Analysis/Normed/Module/Basic.lean,Mathlib/Topology/Bornology/Basic.lean,Mathlib/Topology/Bornology/Constructions.lean,Mathlib/Topology/MetricSpace/Bounded.lean,Mathlib/Topology/MetricSpace/GromovHausdorffRealized.lean 6 1 ['github-actions'] nobody
306-30743
10 months ago
306-30743
10 months ago
0-0
0 seconds
14994 kim-em
author:kim-em
profiling: skipKernelTC merge-conflict 2/1 lakefile.lean 1 3 ['github-actions', 'kim-em', 'leanprover-bot'] nobody
304-62887
10 months ago
304-62887
10 months ago
0-0
0 seconds
15400 grunweg
author:grunweg
feat: "confusing variables" linter This linter flags `variable` commands which both update an existing binder annotation and declare new variables: these can yield confusing or misleading error messages (see leanprover/lean4#2789). Instead, these should be split in several `variable` statements. ---------- Help fixing these errors is welcome! Currently, the linter only catches *some* cases, when the updated binder is from a previous scope. To make it catch all cases, the linter could insert a `section` before the `variable` command and use that scope instead. See [zulip](https://leanprover.zulipchat.com/#narrow/stream/113488-general/topic/Get.20scope.20*before*.20some.20syntax.20is.20evaluated) [discussions](https://leanprover.zulipchat.com/#narrow/stream/113488-general/topic/Determining.20variable.20binders.20from.20syntax). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-linter merge-conflict WIP 292/47 Cache/Requests.lean,Mathlib/Analysis/NormedSpace/OperatorNorm/Prod.lean,Mathlib/Dynamics/Ergodic/Ergodic.lean,Mathlib/FieldTheory/AbelRuffini.lean,Mathlib/FieldTheory/Adjoin.lean,Mathlib/FieldTheory/IntermediateField.lean,Mathlib/FieldTheory/KummerExtension.lean,Mathlib/FieldTheory/Minpoly/MinpolyDiv.lean,Mathlib/FieldTheory/Normal.lean,Mathlib/FieldTheory/PurelyInseparable.lean,Mathlib/Geometry/Manifold/BumpFunction.lean,Mathlib/Geometry/Manifold/ChartedSpace.lean,Mathlib/Geometry/Manifold/ContMDiff/Basic.lean,Mathlib/Geometry/Manifold/PartitionOfUnity.lean,Mathlib/Geometry/Manifold/VectorBundle/Basic.lean,Mathlib/Geometry/Manifold/VectorBundle/Tangent.lean,Mathlib/LinearAlgebra/CliffordAlgebra/Basic.lean,Mathlib/Tactic/Linter/Lint.lean,Mathlib/Tactic/ToAdditive/Frontend.lean,Mathlib/Topology/FiberBundle/Basic.lean,Mathlib/Topology/FiberBundle/Trivialization.lean,test/Lint.lean 22 1 ['github-actions'] nobody
301-23837
9 months ago
306-60859
10 months ago
0-0
0 seconds
10717 joelriou
author:joelriou
feat(Algebra/Homology): the total complex of a tricomplex Given a triple homological complex, there are two ways to obtain a single complex. Under certain assumptions on signs, it is shown in this PR that they are isomorphic. --- - [x] depends on: #10711 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory merge-conflict WIP 968/8 Mathlib.lean,Mathlib/Algebra/Homology/ComplexShapeSigns.lean,Mathlib/Algebra/Homology/HomologicalTricomplex.lean,Mathlib/Algebra/Homology/TotalComplex.lean,Mathlib/Algebra/Homology/TotalComplexShift.lean 5 3 ['github-actions', 'leanprover-community-mathlib4-bot'] nobody
301-19376
9 months ago
301-19376
9 months ago
0-0
0 seconds
12143 adomani
author:adomani
feat: generic linter, absorbing `cdot` linter and `attribute [instance] in` linter A "generic" syntax linter that can be configured using a function `Syntax → Array Syntax`. The expectations is that the function returns sub-syntax extracted from the input that should be flagged by the linter. This PR provides two examples. * Flags uses of `cdot` that are not typed as `·`. * #12137 is a PR that inspired this one. * Flag uses of `attribute [instance] in` that is not limited to the next declaration * Inspired by the existing PR by Michael Rothgang #13190 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-linter merge-conflict 210/2 Mathlib.lean,Mathlib/Combinatorics/Colex.lean,Mathlib/NumberTheory/LegendreSymbol/AddCharacter.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter.lean,Mathlib/Tactic/Linter/GenericSyntaxLinter.lean,test/GenericSyntaxLinter.lean 7 17 ['adomani', 'github-actions', 'grunweg', 'leanprover-bot'] nobody
301-15084
9 months ago
301-15084
9 months ago
41-49960
41 days
14654 grunweg
author:grunweg
feat(runLinter): allow only running certain linters This adds a script `run_linter`, which is a fork of batteries' `runLinter` with extra features: - rewrite as a CLI app, so --help messages etc. come for free - add a `--list` option, which prints the list of linters it was about to run, and exists - add `--select`, `--ignore` and `--only` options which ensure certain linters are always run, never resp. that only a certain list of linters are run. (`add` takes priority over `exclude` or `only`.) - add an `update_only_remove` flag which only runs linters mentioned in the `nolints` file: this only removes entries (by design), but is often much faster. - renamed to `run_linter`: actually, per the [zulip discussion](https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/Naming.20convention/near/450896930), this should be `run-linter` --- and one could as well use the opportunity to rename this to e.g. `env-linter`. Asked [here](https://leanprover.zulipchat.com/#narrow/stream/270676-lean4/topic/Configuring.2Fmodernizing.20runLinter). Intended use cases 1. Run `update_only_remove` when updating the nolints file. In fact, it is so fast that it could even run during regular CI, after the normal `lint` step... 2. Run the mathlib linters locally. The simpNF linters are slow enough (for a reason, but still) that doing so is currently annoying. On my notebook, they can easily take half an hour, during which my notebook is otherwise hardly usable. 3. You're developing a new linter and only want to run *that* one (as there was no change about the other ones). Probably, the nicest result would be this PR landing in batteries (perhaps in pieces) instead of here. --- Two CLI warts I'm unhappy about. - how can I have flag names with a hyphen? Currently, I have to write `--print_linters`, which is less pretty. - many options take an `Array String`: how can I pass this to the executable? This is not obvious to me... [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-linter RFC merge-conflict 320/146 Mathlib/Analysis/LocallyConvex/Bounded.lean,Mathlib/Analysis/Oscillation.lean,Mathlib/Geometry/Manifold/LocalInvariantProperties.lean,Mathlib/MeasureTheory/Measure/EverywherePos.lean,Mathlib/SetTheory/Ordinal/Topology.lean,Mathlib/Topology/Algebra/Group/Basic.lean,Mathlib/Topology/Algebra/Module/Basic.lean,Mathlib/Topology/Algebra/Monoid.lean,Mathlib/Topology/Bases.lean,Mathlib/Topology/Basic.lean,Mathlib/Topology/Category/TopCat/Basic.lean,Mathlib/Topology/Clopen.lean,Mathlib/Topology/CompactOpen.lean,Mathlib/Topology/Compactness/LocallyCompact.lean,Mathlib/Topology/Constructions.lean,Mathlib/Topology/ContinuousOn.lean,Mathlib/Topology/DenseEmbedding.lean,Mathlib/Topology/Gluing.lean,Mathlib/Topology/Homeomorph.lean,Mathlib/Topology/IndicatorConstPointwise.lean,Mathlib/Topology/Inseparable.lean,Mathlib/Topology/Irreducible.lean,Mathlib/Topology/IsLocalHomeomorph.lean,Mathlib/Topology/LocalAtTarget.lean,Mathlib/Topology/Maps/Basic.lean,Mathlib/Topology/MetricSpace/Isometry.lean,Mathlib/Topology/NoetherianSpace.lean,Mathlib/Topology/Order.lean,Mathlib/Topology/Order/LowerUpperTopology.lean,Mathlib/Topology/Partial.lean,Mathlib/Topology/PartialHomeomorph.lean,Mathlib/Topology/PartitionOfUnity.lean,Mathlib/Topology/QuasiSeparated.lean,Mathlib/Topology/Separation.lean,Mathlib/Topology/TietzeExtension.lean,Mathlib/Topology/UniformSpace/Ascoli.lean,Mathlib/Topology/UniformSpace/Basic.lean,Mathlib/Topology/UniformSpace/Cauchy.lean,Mathlib/Topology/UniformSpace/CompactConvergence.lean,Mathlib/Topology/UniformSpace/Completion.lean,Mathlib/Topology/UniformSpace/Equicontinuity.lean,Mathlib/Topology/UniformSpace/Matrix.lean,Mathlib/Topology/UniformSpace/Pi.lean,Mathlib/Topology/UnitInterval.lean,Mathlib/Topology/UrysohnsBounded.lean,Mathlib/Topology/UrysohnsLemma.lean,Mathlib/Topology/VectorBundle/Basic.lean,lakefile.lean,scripts/run_linter.lean 49 5 ['github-actions', 'grunweg', 'rosborn'] nobody
301-687
9 months ago
301-687
9 months ago
13-61906
13 days
15679 adomani
author:adomani
test: refactor in CI --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP 213/5 .github/workflows/bors.yml,.github/workflows/build.yml,.github/workflows/build.yml.in,.github/workflows/build_fork.yml,Mathlib.lean,Mathlib/Algebra/Homology/HomotopyCategory/SingleFunctors.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Affine.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Order.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Unique.lean,Mathlib/Analysis/Convex/Combination.lean,Mathlib/Analysis/Convex/Segment.lean,Mathlib/CategoryTheory/Bicategory/Adjunction.lean,Mathlib/CategoryTheory/Monoidal/Braided/Basic.lean,Mathlib/CategoryTheory/Monoidal/Center.lean,Mathlib/GroupTheory/Coxeter/Matrix.lean,Mathlib/Order/Filter/Cocardinal.lean,Mathlib/Order/UpperLower/Basic.lean,Mathlib/TestRefactor.lean,Refactor/Main.lean,lakefile.lean,lean-toolchain 21 1 ['github-actions'] nobody
300-86319
9 months ago
300-86319
9 months ago
0-8
8 seconds
7565 shuxuezhuyi
author:shuxuezhuyi
feat(Topology/Algebra/Order): extend homeomorphism of `Ioo` to `Icc` We extend the homeomorphisms between open intervals to homeomorphisms between the closed intervals. --- - [ ] depends on: #7018 - [ ] depends on: #7351 - [ ] depends on: #7564 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order t-topology merge-conflict blocked-by-other-PR 389/5 Mathlib.lean,Mathlib/Data/Set/Intervals/Image.lean,Mathlib/Order/Directed.lean,Mathlib/Topology/Algebra/Order/IccExtendFromIoo.lean,Mathlib/Topology/Algebra/Order/IntermediateValue.lean 5 1 ['leanprover-community-mathlib4-bot'] nobody
299-36419
9 months ago
299-36419
9 months ago
0-0
0 seconds
10629 madvorak
author:madvorak
feat: List.cons_sublist_append_iff_right --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data merge-conflict 11/0 Mathlib/Data/List/Basic.lean 1 1 ['eric-wieser'] nobody
299-36310
9 months ago
299-36310
9 months ago
53-73442
53 days
9973 Ruben-VandeVelde
author:Ruben-VandeVelde
feat: polynomials formed by lists From https://github.com/leanprover-community/mathlib/pull/15476 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data merge-conflict please-adopt 311/0 Mathlib.lean,Mathlib/Data/Polynomial/OfList.lean 2 0 [] nobody
299-35843
9 months ago
299-35843
9 months ago
0-0
0 seconds
12926 joelriou
author:joelriou
feat(CategoryTheory): the monoidal category structure induced by a monoidal functor In this PR, given a monoidal functor `F : MonoidalFunctor C D`, we define a monoidal category structure on the category `InducedCategory D F.obj`, which has the "same" objects as `C`, but the morphisms between `X` and `Y` identify to `F.obj X ⟶ F.obj Y`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory merge-conflict WIP 105/0 Mathlib.lean,Mathlib/CategoryTheory/Monoidal/Induced.lean 2 3 ['eric-wieser', 'github-actions', 'joelriou'] nobody
299-34242
9 months ago
299-34242
9 months ago
0-0
0 seconds
12869 adomani
author:adomani
feat: linter and script for `theorem` vs `lemma` This PR contains a linter for flagging doc-string-less `theorem`s, as well as a bash script that, once the linter ran on Mathlib, automatically replaces every linter-offending `theorem` by `lemma`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-linter merge-conflict awaiting-author 106/0 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter/ThmLemma.lean,scripts/thmLemma.sh 4 13 ['adomani', 'github-actions', 'grunweg', 'joneugster'] nobody
299-21006
9 months ago
299-21006
9 months ago
0-0
0 seconds
14308 grhkm21
author:grhkm21
feat(Algebra/Category): Direct construction of colimits in algebraic categories (Below I only write about colimits since that's what I'm familiar with after working on it the last few days, but maybe it's the same for other categorical constructions) **Main feature:** Construct colimits in `AddCommGrp`/`ModuleCat`/`FGModuleCat`(/...) directly as coequalizer (i.e. cokernel i.e. quotient) of two maps, allowing one to say $\coprod_j M_j \cong *$ Currently, if you look at how colimits are constructed for [AddCommGrp](https://github.com/leanprover-community/mathlib4/blob/master/Mathlib/Algebra/Category/Grp/Colimits.lean#L69-L92), you see this massive block of code of all relations generating the quotient relation, but that's kind of bad, you can't say anything concretely about it. Also as noted in the TODOs of a few files: ``` TODO: In fact, in `ModuleCat R` there is a much nicer model of colimits as quotients of finitely supported functions, and we really should implement this as well. ``` I wrote it down [here](https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/Braided.20left.20rigid.20categories.20are.20right.20rigid/near/447490672), and **have formalised it** in a small file already [here](https://gist.github.com/grhkm21/5b2d938753c0ce0900d21c93a39e3b7d#file-addcommgrpcolimits-lean-L162-L163) (I also have a `ModuleCat` version, and proving existence of colimits in `FGModuleCat` from it). Usually I will try to merge the file into Mathlib directly (preferably in one sitting), but I have been trying for a while now and been struggling. One issue is I am struggling to understand universes, which I asked [here](https://leanprover.zulipchat.com/#narrow/stream/113489-new-members/topic/Universe.20constraints!/near/448049266) along with many other places. A more concrete issue is that - [ ] FGModuleCat (and `FullSubcategory` in general) requires morphism and objects to be on the same universe, whereas generally `Category.{v, u}` don't. So that seems to limit what I can express, and maybe I have to fix it first. Here are a few more TODOs just so I don't forget, probably done before the one above: - [ ] Generalise `cokernelIsoQuotient` to other categories. - [ ] Also prove `coproductIsoDirectSum` - [ ] Also prove coequalizer (f + h) (g + h) ~ coequalizer f g ~ cokernel (f - g) 0 - [ ] Fix typo `FGModuleCatCat` If anyone is familiar with universe stuff and can answer my many questions that'll be great too. I need help understanding just [these five lines](https://github.com/leanprover-community/mathlib4/blob/master/Mathlib/Algebra/Category/Grp/Colimits.lean#L267-L271) t-algebra merge-conflict WIP
label:t-algebra$
10/3 Mathlib/Algebra/DirectSum/Module.lean,Mathlib/LinearAlgebra/FreeModule/Basic.lean 2 1 ['github-actions'] nobody
298-33027
9 months ago
298-33027
9 months ago
0-0
0 seconds
12695 chrisflav
author:chrisflav
feat(RingTheory/Smooth): smooth morphisms are flat We show that smooth ring homomorphisms are flat. The strategy for a smooth `A`-algebra `B` is the following: - first we find a model of `B` over a Noetherian base ring - if `A` is Noetherian, we identify `B` as a retract of the adic completion of a polynomial ring over `A`, which is flat This is the summary PR which will be split in several parts. Co-authored-by: Judith Ludwig --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict
label:t-algebra$
2767/1 Mathlib.lean,Mathlib/Algebra/DirectSum/Basic.lean,Mathlib/Algebra/Exact.lean,Mathlib/Algebra/Module/Torsion.lean,Mathlib/LinearAlgebra/SModEq.lean,Mathlib/RingTheory/AdicCompletion/Algebra.lean,Mathlib/RingTheory/AdicCompletion/AsTensorProduct.lean,Mathlib/RingTheory/AdicCompletion/Basic.lean,Mathlib/RingTheory/AdicCompletion/Exactness.lean,Mathlib/RingTheory/AdicCompletion/Functoriality.lean,Mathlib/RingTheory/RingOfDefinition.lean,Mathlib/RingTheory/RingOfDefinition/RingModel.lean,Mathlib/RingTheory/RingOfDefinition/Utils.lean,Mathlib/RingTheory/RingOfDefinitionIdeal.lean,Mathlib/RingTheory/Smooth/Descent.lean,Mathlib/RingTheory/Smooth/Flat.lean 16 0 [] nobody
298-32942
9 months ago
298-32942
9 months ago
0-0
0 seconds
12744 chrisflav
author:chrisflav
feat(RingTheory/Smooth): Noetherian ring of definition We show that given a smooth `A`-algebra `B`, there exists a subring `A₀` of `A` of finite type over `ℤ` and a smooth `A₀`-algebra `B₀` such that `B = A ⊗[A₀] B₀`. A reference is https://stacks.math.columbia.edu/tag/00TP. This is also a test case for the ring of definition API. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict
label:t-algebra$
1212/0 Mathlib/Algebra/Algebra/Hom.lean,Mathlib/Algebra/MvPolynomial/Basic.lean,Mathlib/RingTheory/FiniteType.lean,Mathlib/RingTheory/Ideal/Operations.lean,Mathlib/RingTheory/MvPolynomial/Homogeneous.lean,Mathlib/RingTheory/RingOfDefinition/BaseChange.lean,Mathlib/RingTheory/RingOfDefinition/Basic.lean,Mathlib/RingTheory/RingOfDefinition/Relations.lean,Mathlib/RingTheory/Smooth/Descent.lean,Mathlib/ToBeMoved.lean 10 0 [] nobody
298-32941
9 months ago
298-32941
9 months ago
0-0
0 seconds
12743 chrisflav
author:chrisflav
feat(RingTheory/RingOfDefinition): basic API Given a finitely presented algebra `A` over a ring `R`, we may descend to a Noetherian subring `R₀` of `R` and a model of `A` over `R₀`. In this PR we provide basic API for working with polynomial rings over subrings. In particular we provide infrastructure for producing `R₀` and descending polynomials in `R` to polynomials in `R₀` given containment of the coefficients. Notation: `R` is a ring, `R₀` a subring, `p : MvPolynomial ι R` and `s : Set (MvPolynomial ι R)`. ## Main definitions For producing subrings containing a set of polynomials of interest, we provide the following: - `HasCoefficients p R₀`: typeclass expressing that the coefficients of `p` are contained in `R₀`. - `core s`: adjoin the coefficients of a set of polynomials `s` to `ℤ`. - `adjoinCoefficients s R₀`: adjoin the coefficients of a set of polynomials `s` to `R₀`. - `repr p R₀`: Given `[HasCoefficients p R₀]` and a polynomial `p`, this is the representative of `p` as a polynomial over `R₀`. Instances for `HasCoefficients` are provided to ensure that the following facts are automatically inferred: - the coefficients of any polynomial in `s` are contained in `core s`. - if the coefficients of `p` are in `R₀` and we adjoin the coefficients of `s`, then the coefficients of `p` are also in `adjoinCoefficients s R₀`. Now, given a (finitely) presented `R` algebra, expressed through an ideal `I : Ideal R`, a `Model` of `I` is a structure containing - a set `s` of generators of `I` - a subring `R₀` - a proof that the coefficients of `s` are contained in `R₀` Given such a model `M`, we expose: - `M.s₀`: the intersection of `s` with `MvPolynomial ι R₀`. Informally this is simply `s`. - `M.I₀`: the ideal generated by `M.s₀` - `M.A₀`: the quotient `MvPolynomial ι M.R₀ ⧸ MvPolynomial ι M.I₀` In `RingOfDefinition/BaseChange` we show that `R ⊗[R₀] M.A₀` is `R`-isomorphic to `MvPolynomial ι R ⧸ I` (this is done in a more general setting and then specialized to this situation). Since `M.I₀` is not equal to `I` intersected with `R₀`, more technical difficulties arise. To work around these, we introduce - `Relation A`: For an arbitrary `A : Set R`, this is simply `MvPolynomial A R`. In the following we are particularly interested in the case where `A = s = Set (MvPolynomial ι R)` is a set of generators of `I`. An equation `x = y` in `MvPolynomial ι R ⧸ I` can be expressed as `x - y ∈ I`. In this case there exists a `r : Relation s` such that `eval r = x - y`. Here `eval` is a shortcut for `MvPolynomial.eval Subtype.val`, i.e. we evaluate the formal expression `r` in the ring `MvPolynomial ι R`. To preserve this equation in `MvPolynomial ι R₀ ⧸ I₀`, we need to adjoin the coefficients of `r` to `R₀`. For this a similar API is provided, in particular: - `HasRelation r R₀`: a typeclass expressing that the coefficients of `r` are contained in `R₀`. - `adjoinRelations rs R₀`: adjoin the coefficients of a set of relations to `R₀`. - `repr r M`: Given `[HasRelation r M.R₀]`, this is the representative of `r` over `R₀`, i.e. an element of `Relation M.s₀` that is mapped to `r` under the canonical map `Relation M.s₀ → Relation M.s`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict
label:t-algebra$
797/0 Mathlib/Algebra/Algebra/Hom.lean,Mathlib/Algebra/MvPolynomial/Basic.lean,Mathlib/RingTheory/FiniteType.lean,Mathlib/RingTheory/Ideal/Operations.lean,Mathlib/RingTheory/MvPolynomial/Homogeneous.lean,Mathlib/RingTheory/RingOfDefinition/BaseChange.lean,Mathlib/RingTheory/RingOfDefinition/Basic.lean 7 0 [] nobody
298-32941
9 months ago
298-32941
9 months ago
0-0
0 seconds
13010 ADedecker
author:ADedecker
feat: relax universe constraint in stoneCechExtend --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology merge-conflict 33/3 Mathlib/Topology/StoneCech.lean 1 2 ['ADedecker', 'erdOne'] nobody
298-32824
9 months ago
298-32824
9 months ago
0-0
0 seconds
12411 adomani
author:adomani
feat: more linting of cdots --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-linter merge-conflict 953/617 Archive/Wiedijk100Theorems/CubingACube.lean,Mathlib.lean,Mathlib/Algebra/Category/GroupCat/Colimits.lean,Mathlib/Algebra/Homology/Exact.lean,Mathlib/Algebra/Homology/LocalCohomology.lean,Mathlib/Algebra/Lie/Nilpotent.lean,Mathlib/Algebra/Module/PID.lean,Mathlib/Algebra/Module/Submodule/Bilinear.lean,Mathlib/Algebra/Module/Torsion.lean,Mathlib/Algebra/MonoidAlgebra/Basic.lean,Mathlib/Algebra/Order/Archimedean.lean,Mathlib/AlgebraicGeometry/StructureSheaf.lean,Mathlib/Analysis/Analytic/Composition.lean,Mathlib/Analysis/Calculus/Deriv/Slope.lean,Mathlib/Analysis/Calculus/InverseFunctionTheorem/ApproximatesLinearOn.lean,Mathlib/Analysis/Calculus/LocalExtr/Basic.lean,Mathlib/Analysis/Calculus/TangentCone.lean,Mathlib/Analysis/InnerProductSpace/Basic.lean,Mathlib/Analysis/InnerProductSpace/Projection.lean,Mathlib/Analysis/MeanInequalitiesPow.lean,Mathlib/Analysis/Normed/Group/ControlledClosure.lean,Mathlib/Analysis/Normed/Group/Pointwise.lean,Mathlib/Analysis/NormedSpace/FiniteDimension.lean,Mathlib/Analysis/NormedSpace/HahnBanach/Separation.lean,Mathlib/Analysis/NormedSpace/Multilinear/Basic.lean,Mathlib/Analysis/NormedSpace/Star/Basic.lean,Mathlib/Analysis/NormedSpace/Star/Multiplier.lean,Mathlib/Analysis/NormedSpace/lpSpace.lean,Mathlib/Analysis/PSeries.lean,Mathlib/Analysis/RCLike/Basic.lean,Mathlib/Analysis/SpecialFunctions/Complex/Arg.lean,Mathlib/Analysis/SpecialFunctions/Log/Base.lean,Mathlib/Analysis/SpecialFunctions/Log/Monotone.lean,Mathlib/Analysis/SpecialFunctions/Pow/NNReal.lean,Mathlib/Analysis/SpecialFunctions/Pow/Real.lean,Mathlib/Analysis/SpecificLimits/Normed.lean,Mathlib/CategoryTheory/Abelian/Basic.lean,Mathlib/CategoryTheory/Action.lean,Mathlib/CategoryTheory/Bicategory/NaturalTransformation.lean,Mathlib/CategoryTheory/Category/Cat/Limit.lean,Mathlib/CategoryTheory/Category/PartialFun.lean,Mathlib/CategoryTheory/Category/TwoP.lean,Mathlib/CategoryTheory/Closed/Cartesian.lean,Mathlib/CategoryTheory/Functor/Flat.lean,Mathlib/CategoryTheory/Galois/GaloisObjects.lean,Mathlib/CategoryTheory/Limits/Over.lean,Mathlib/CategoryTheory/Limits/VanKampen.lean,Mathlib/CategoryTheory/Localization/Predicate.lean,Mathlib/CategoryTheory/Monad/Coequalizer.lean,Mathlib/CategoryTheory/Monad/Monadicity.lean,Mathlib/CategoryTheory/Pi/Basic.lean,Mathlib/CategoryTheory/Sites/DenseSubsite.lean,Mathlib/CategoryTheory/Sites/InducedTopology.lean,Mathlib/CategoryTheory/Subobject/Lattice.lean,Mathlib/Combinatorics/Additive/PluenneckeRuzsa.lean,Mathlib/Combinatorics/HalesJewett.lean,Mathlib/Combinatorics/SimpleGraph/Regularity/Chunk.lean,Mathlib/Computability/Reduce.lean,Mathlib/Data/Holor.lean,Mathlib/Data/Nat/Multiplicity.lean,Mathlib/Data/Nat/Pairing.lean,Mathlib/Data/Real/Cardinality.lean,Mathlib/Data/Real/Hyperreal.lean,Mathlib/Data/Real/Irrational.lean,Mathlib/Data/Set/Card.lean,Mathlib/Dynamics/Circle/RotationNumber/TranslationNumber.lean,Mathlib/FieldTheory/Finite/Polynomial.lean,Mathlib/FieldTheory/Minpoly/IsIntegrallyClosed.lean,Mathlib/FieldTheory/PerfectClosure.lean,Mathlib/FieldTheory/RatFunc.lean,Mathlib/Geometry/RingedSpace/OpenImmersion.lean,Mathlib/Geometry/RingedSpace/PresheafedSpace/Gluing.lean,Mathlib/GroupTheory/GroupAction/Quotient.lean,Mathlib/GroupTheory/Nilpotent.lean,Mathlib/GroupTheory/Perm/Cycle/Factors.lean,Mathlib/GroupTheory/Perm/Finite.lean,Mathlib/GroupTheory/SpecificGroups/Quaternion.lean,Mathlib/GroupTheory/Sylow.lean,Mathlib/LinearAlgebra/Dimension/RankNullity.lean,Mathlib/LinearAlgebra/Dual.lean,Mathlib/LinearAlgebra/LinearIndependent.lean,Mathlib/LinearAlgebra/LinearPMap.lean,Mathlib/LinearAlgebra/Matrix/Charpoly/Coeff.lean,Mathlib/LinearAlgebra/Prod.lean,Mathlib/LinearAlgebra/QuadraticForm/Complex.lean,Mathlib/LinearAlgebra/Reflection.lean,Mathlib/MeasureTheory/Constructions/Pi.lean,Mathlib/MeasureTheory/Covering/VitaliFamily.lean,Mathlib/MeasureTheory/Measure/Haar/Basic.lean,Mathlib/MeasureTheory/Measure/MeasureSpace.lean,Mathlib/MeasureTheory/Measure/Typeclasses.lean,Mathlib/MeasureTheory/OuterMeasure/Basic.lean,Mathlib/ModelTheory/Skolem.lean,Mathlib/NumberTheory/Dioph.lean,Mathlib/NumberTheory/LegendreSymbol/Basic.lean,Mathlib/NumberTheory/Padics/Hensel.lean,Mathlib/NumberTheory/Padics/PadicNumbers.lean,Mathlib/NumberTheory/Padics/RingHoms.lean,Mathlib/NumberTheory/RamificationInertia.lean,Mathlib/RingTheory/AdjoinRoot.lean 147 2 ['adomani', 'leanprover-bot'] nobody
298-32687
9 months ago
298-32687
9 months ago
0-0
0 seconds
12279 casavaca
author:casavaca
WIP: feat: Holder's inequality n-ary --- - [x] depends on #12291 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis merge-conflict WIP 129/0 Mathlib/Analysis/MeanInequalities.lean,Mathlib/Analysis/SpecialFunctions/Pow/Real.lean 2 13 ['github-actions'] nobody
298-32672
9 months ago
298-32672
9 months ago
0-0
0 seconds
12093 ADedecker
author:ADedecker
feat: tweak the definition of semicontinuity to behave better in nonlinear orders Summary of the changes: - change definitions to make [lowerSemicontinuous_iff_isClosed_preimage](https://leanprover-community.github.io/mathlib4_docs/Mathlib/Topology/Semicontinuous.html#lowerSemicontinuous_iff_isClosed_preimage) true without assuming `LinearOrder`, so that semicontinuity corresponds to continuity for lower/upper order topology on the codomain. See discussion on [Zulip](https://leanprover.zulipchat.com/#narrow/stream/116395-maths/topic/Semicontinuity.20definition.20for.20non-linear.20orders/near/432898278) - add new `iff` lemmas for unfolding the definition - add `iff` lemmas with the old definition in the linearly ordered case - some basic lemmas need to be changed in an easy way - minimize assumptions for continuity => semicontinuity - prove the semicontinuity criterion for indicators using "preimage of Ici/Iic" instead of a direct proof, because the proof is more natural (especially because we have no `filter_upwards` for `Frequently`) - in the rest of the file (which is about linear orders anyway), we don't touch the statements and just rewrite to the old definition. Some of these could be generalized, but we keep that for a later PR. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology merge-conflict WIP 274/130 Mathlib/Analysis/BoundedVariation.lean,Mathlib/MeasureTheory/Integral/FundThmCalculus.lean,Mathlib/Order/Filter/Basic.lean,Mathlib/Topology/Semicontinuous.lean 4 0 [] nobody
298-32634
9 months ago
298-32634
9 months ago
0-0
0 seconds
11520 thorimur
author:thorimur
feat: `linting_rules` and deprecated syntax --- Experimental. WIP. Might not be performance-viable. - [ ] depends on: #11519 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta merge-conflict blocked-by-other-PR 1016/0 Mathlib.lean,Mathlib/Command/Linter.lean,Mathlib/Command/Linter/Deprecated.lean,Mathlib/Command/Linter/LintingRules.lean,Mathlib/Command/SyntaxRules.lean,Mathlib/Command/SyntaxRules/Attr.lean,Mathlib/Command/SyntaxRules/Elab.lean,Mathlib/Command/SyntaxRules/Header.lean,Mathlib/Command/SyntaxRules/Util.lean,Mathlib/Tactic/Common.lean,scripts/noshake.json 11 11 ['leanprover-bot', 'leanprover-community-mathlib4-bot', 'thorimur'] nobody
298-32624
9 months ago
298-32624
9 months ago
0-0
0 seconds
11519 thorimur
author:thorimur
feat: `syntax_rules` --- Experimental. WIP. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta merge-conflict 485/0 Mathlib.lean,Mathlib/Command/SyntaxRules.lean,Mathlib/Command/SyntaxRules/Attr.lean,Mathlib/Command/SyntaxRules/Elab.lean,Mathlib/Command/SyntaxRules/Header.lean,Mathlib/Command/SyntaxRules/Util.lean,scripts/noshake.json 7 0 [] nobody
298-32610
9 months ago
298-32610
9 months ago
0-0
0 seconds
11393 mcdoll
author:mcdoll
feat(Analysis/Distribution/SchwartzSpace): The Heine-Borel property --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis merge-conflict WIP 688/3 Mathlib.lean,Mathlib/Analysis/Distribution/SchwartzSpace.lean,Mathlib/Topology/Constructions.lean,Mathlib/Topology/UniformSpace/Ascoli.lean,Mathlib/Topology/UniformSpace/Pi.lean,Mathlib/Topology/UniformSpace/UniformConvergenceTopology.lean 6 0 [] nobody
298-32600
9 months ago
298-32600
9 months ago
0-0
0 seconds
12310 BoltonBailey
author:BoltonBailey
feat: add Tropically bound polynomials Co-authored-by: Junyan Xu --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra awaiting-CI merge-conflict awaiting-author
label:t-algebra$
31/0 Mathlib.lean,Mathlib/Algebra/Tropical/TropicallyBoundPolynomial/Basic.lean 2 0 [] nobody
298-32561
9 months ago
298-32561
9 months ago
0-0
0 seconds
9444 erdOne
author:erdOne
feat: Various instances regarding `𝓞 K`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-number-theory merge-conflict help-wanted 27/0 Mathlib/NumberTheory/NumberField/Basic.lean,Mathlib/RingTheory/IntegralClosure.lean 2 9 ['erdOne', 'leanprover-bot', 'mattrobball', 'riccardobrasca', 'xroblot'] nobody
298-32519
9 months ago
298-32519
9 months ago
0-0
0 seconds
8931 hmonroe
author:hmonroe
feat(Computable): define P, NP, and NP-complete Revised to focus on languages that are binary strings, given the issue of non-acceptable encodings of unspecified Types --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-computability merge-conflict awaiting-author 381/5 Mathlib.lean,Mathlib/Computability/Complexity copy.lean,Mathlib/Computability/Complexity.lean,Mathlib/Computability/Encoding.lean,Mathlib/Computability/TMComputable.lean,Mathlib/Computability/TuringMachine.lean,Mathlib/Computability/halting example.lean,docs/references.bib 8 3 ['fpvandoorn', 'github-actions', 'hmonroe'] nobody
298-32484
9 months ago
298-32484
9 months ago
5-62479
5 days
10641 newell
author:newell
feat(Topology/MetricSpace/WellSpaced): Define sets that are *well-spaced*. Create a new file `Mathlib.Topology.MetricSpace.WellSpaced` that contains definitions of sets which are in some sense *well-spaced*. Some examples are Delone and Meyer sets, which find applications in Quasicrystals and Coding Theory, among others. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology merge-conflict 1073/14 Mathlib.lean,Mathlib/Analysis/LocallyConvex/WithSeminorms.lean,Mathlib/Topology/EMetricSpace/Basic.lean,Mathlib/Topology/GMetric/Basic.lean,Mathlib/Topology/GMetric/GInfSep.lean,Mathlib/Topology/GMetric/WellSpaced.lean,Mathlib/Topology/GPseudoMetric/Basic.lean,Mathlib/Topology/MetricSpace/WellSpaced.lean 8 1 ['edegeltje'] nobody
298-32452
9 months ago
298-32452
9 months ago
0-0
0 seconds
10428 dwrensha
author:dwrensha
feat: add simp_digits tactic With the introduction of the simprocs `reduceLE`, `reduceMod`, `reduceDiv` etc. in Lean v4.6.0, now `simp` can fully normalize typical `Nat.digits` calls that have concrete arguments. The situation is still a bit delicate however, as we want to avoid invoking kernel reduction on `Nat.digits`, because the `Acc`-based ("well founded") recursion in `digitsAux` can get bogged down. This PR introduces a new tactic `simp_digits` tactic that contains only the simp lemmas and simprocs needed to reduce `Nat.digits`. This allows proofs involving `Nat.digits` to be cleanly factored into two steps: 1. reduce `Nat.digits` via `simp_digits`, 2. do things that require kernel reduction such as `simp_arith`, `decide`, or `rfl`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta merge-conflict 6/124 Archive/Imo/Imo1960Q1.lean,Archive/Imo/Imo1962Q1.lean,Mathlib/Data/Nat/Digits.lean 3 2 ['dwrensha'] nobody
298-32306
9 months ago
298-32306
9 months ago
0-0
0 seconds
10345 newell
author:newell
feat(Algebra.Module.Zlattice): Add Voronoi Domain Adds the definition for a Voronoi Domain in regards to the $\mathbb{Z}$-lattice: $$C := \lbrace\mathbf{w} \in \mathbb{V}^n\ :\ |\mathbf{w}| \leq |\mathbf{w} - \mathbf{v}|\ \text{for all}\ \mathbf{v} \in \mathbf{L} \rbrace$$ where $\mathbf{L}\$ is the $\mathbb{Z}$-lattice. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict WIP
label:t-algebra$
17/0 Mathlib/Algebra/Module/Zlattice.lean 1 3 ['alreadydone', 'newell'] nobody
298-32248
9 months ago
298-32248
9 months ago
0-0
0 seconds
8608 eric-wieser
author:eric-wieser
feat: multiplicativize `AddTorsor` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict WIP
label:t-algebra$
268/199 Mathlib/Algebra/AddTorsor.lean,Mathlib/Algebra/Group/Defs.lean,Mathlib/Data/Set/Pointwise/SMul.lean,Mathlib/Tactic/ToAdditive.lean 4 0 [] nobody
298-32129
9 months ago
298-32129
9 months ago
0-0
0 seconds
9154 FR-vdash-bot
author:FR-vdash-bot
feat: `npow` / `nsmul` / `Nat.cast`/ `zpow` / `zsmul` implemented using `Nat.binaryRec` --- - [ ] depends on: https://github.com/leanprover/lean4/pull/3756 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict awaiting-author blocked-by-other-PR
label:t-algebra$
168/359 Mathlib/Algebra/Group/Defs.lean,Mathlib/Computability/PartrecCode.lean,Mathlib/Computability/Primrec.lean,Mathlib/Data/Bool/Basic.lean,Mathlib/Data/Int/Bitwise.lean,Mathlib/Data/Nat/Bits.lean,Mathlib/Data/Nat/Bitwise.lean,Mathlib/Data/Nat/Digits.lean,Mathlib/Data/Nat/EvenOddRec.lean,Mathlib/Data/Nat/Fib/Basic.lean,Mathlib/Data/Nat/Multiplicity.lean,Mathlib/Data/Nat/Order/Basic.lean,Mathlib/Data/Nat/Parity.lean,Mathlib/Data/Nat/Size.lean,Mathlib/Data/Num/Lemmas.lean,Mathlib/Init/Data/Nat/Bitwise.lean,Mathlib/LinearAlgebra/TensorProduct/Graded/Internal.lean,Mathlib/Logic/Basic.lean,Mathlib/Logic/Denumerable.lean,Mathlib/Logic/Encodable/Basic.lean,Mathlib/Logic/Equiv/Basic.lean,Mathlib/Logic/Equiv/Nat.lean,lake-manifest.json,lakefile.lean,test/zmod.lean 25 7 ['FR-vdash-bot', 'eric-wieser', 'kim-em', 'leanprover-community-mathlib4-bot'] nobody
298-32097
9 months ago
298-32097
9 months ago
0-0
0 seconds
6603 tydeu
author:tydeu
feat: automatically try `cache get` before build --- A quick proof-of-concept. With this, `lake build` will always try `cache get` before building mathlib. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) CI merge-conflict WIP 29/0 lakefile.lean 1 3 ['kim-em', 'tydeu'] nobody
298-32071
9 months ago
298-32071
9 months ago
11-1960
11 days
7026 mo271
author:mo271
feat: toMonoidHom_coe - [ ] depends on: #6791 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-number-theory merge-conflict blocked-by-other-PR 16/0 Mathlib/NumberTheory/LegendreSymbol/MulCharacter.lean 1 3 ['leanprover-community-mathlib4-bot', 'mo271'] nobody
298-32060
9 months ago
298-32060
9 months ago
0-0
0 seconds
6058 apurvnakade
author:apurvnakade
feat: duality theory for cone programs This PR tracks the development of duality theory for cone programs. [Reference](https://ti.inf.ethz.ch/ew/courses/ApproxSDP09/notes/conelp.pdf) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) - [x] depends on: #6059 - [ ] define direct sum of cones - [ ] weak duality - [ ] regular duality - [ ] slater condition - [ ] strong duality t-analysis merge-conflict WIP 159/0 Mathlib.lean,Mathlib/Analysis/Convex/Cone/ConeLinearProgram.lean 2 1 ['leanprover-community-mathlib4-bot'] nobody
298-32016
9 months ago
298-32016
9 months ago
0-0
0 seconds
6449 ADedecker
author:ADedecker
feat: functions with finite fibers --- This has been discussed before on [Zulip](https://leanprover.zulipchat.com/#narrow/stream/217875-Is-there-code-for-X.3F/topic/.E2.9C.94.20Cofinite.20maps.3F) and it came up again while working with @kkytola's student. As explained in the docstring, we could absolutely just use `Tendsto f cofinite cofinite` all the time, but (1) we lack some API for it (2) the API is nicer to setup if we have a separate def (e.g for dot notation) and (3) mentioning filters for such a simple concept is really not beginner-friendly. I'm not sure at all about the name. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology merge-conflict awaiting-author 203/0 Mathlib.lean,Mathlib/Logic/Function/HasFiniteFibers.lean,Mathlib/Order/Filter/Basic.lean,Mathlib/Order/Filter/Cofinite.lean 4 14 ['ADedecker', 'YaelDillies', 'alexjbest', 'kkytola'] nobody
298-32010
9 months ago
298-32010
9 months ago
6-70040
6 days
8195 newell
author:newell
Feat (GroupTheory.SpecificGroups.PresentedDihedral): Add a group presentation of the `DihedralGroup n`. Add group presentation $\< a, b\ |\ a ^ 2 = 1, b ^ 2 = 1, (a * b) ^ n = 1 \>$ for `DihedralGroup n`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict WIP
label:t-algebra$
206/2 Mathlib/GroupTheory/PresentedGroup.lean,Mathlib/GroupTheory/SpecificGroups/Dihedral.lean 2 6 ['kbuzzard', 'newell'] nobody
298-31884
9 months ago
298-31884
9 months ago
0-0
0 seconds
8100 digama0
author:digama0
feat: add support for other types in norm_num --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta merge-conflict 177/12 Mathlib/Tactic/NormNum/Basic.lean,Mathlib/Tactic/NormNum/Eq.lean,Mathlib/Tactic/NormNum/Ineq.lean,Mathlib/Tactic/NormNum/Pow.lean,Mathlib/Tactic/NormNum/Result.lean,Mathlib/Tactic/NormNum/Structural.lean,test/norm_num.lean 7 4 ['dwrensha'] nobody
298-31878
9 months ago
298-31878
9 months ago
0-0
0 seconds
7739 mcdoll
author:mcdoll
feat(LinearAlgebra/LinearPMap): difference of inverses --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict WIP
label:t-algebra$
126/7 Mathlib/LinearAlgebra/LinearPMap.lean,lean-toolchain 2 2 ['digama0', 'eric-wieser'] nobody
298-31850
9 months ago
298-31850
9 months ago
0-0
0 seconds
15586 FR-vdash-bot
author:FR-vdash-bot
test make `HasQuotient` out put a `setoid` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict
label:t-algebra$
22/36 Mathlib/Algebra/Lie/CartanExists.lean,Mathlib/Algebra/Lie/Quotient.lean,Mathlib/Algebra/Lie/Weights/Basic.lean,Mathlib/Algebra/Quotient.lean,Mathlib/Analysis/Normed/Group/AddCircle.lean,Mathlib/GroupTheory/Commensurable.lean,Mathlib/GroupTheory/Coset.lean,Mathlib/GroupTheory/CosetCover.lean,Mathlib/GroupTheory/GroupAction/Quotient.lean,Mathlib/GroupTheory/Nilpotent.lean,Mathlib/GroupTheory/QuotientGroup.lean,Mathlib/LinearAlgebra/Quotient.lean,Mathlib/RingTheory/Ideal/Quotient.lean,Mathlib/Topology/Algebra/UniformRing.lean 14 5 ['FR-vdash-bot', 'github-actions', 'leanprover-bot'] nobody
296-64286
9 months ago
296-64286
9 months ago
0-0
0 seconds
15585 FR-vdash-bot
author:FR-vdash-bot
test make `HasQuotient.quotient'` reducible --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict
label:t-algebra$
8/1 Mathlib/Algebra/Quotient.lean,Mathlib/GroupTheory/Coset.lean 2 1 ['github-actions'] nobody
296-64286
9 months ago
296-64286
9 months ago
0-0
0 seconds
11632 mattrobball
author:mattrobball
chore(Group/RingTheory.Congruence): make `Quotient`'s reducible These are essentially wrappers and should not expose any data when made reducible. Their use in constructing typeclass instances makes reducible transparency desirable. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict 16/35 Mathlib/GroupTheory/Congruence/Basic.lean,Mathlib/RingTheory/Congruence/Basic.lean 2 14 ['eric-wieser', 'fpvandoorn', 'github-actions', 'grunweg', 'kmill', 'leanprover-bot', 'mattrobball'] nobody
294-85734
9 months ago
325-21094
10 months ago
2-10495
2 days
13791 digama0
author:digama0
refactor: Primrec and Partrec General cleanup of the `Primrec` and `Partrec` files, to better adjust to lean 4 things. The main user-visible change is that `Primrec₂` is no longer a `def` but an `abbrev`, because it was causing inference issues in lean 4. I also removed all the nonterminal `simp`s in `PartrecCode.lean`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) tech debt t-computability merge-conflict 585/778 Mathlib/Computability/Ackermann.lean,Mathlib/Computability/Halting.lean,Mathlib/Computability/Partrec.lean,Mathlib/Computability/PartrecCode.lean,Mathlib/Computability/Primrec.lean 5 2 ['github-actions', 'grunweg'] nobody
294-85555
9 months ago
335-23470
11 months ago
1-84718
1 day
11964 adamtopaz
author:adamtopaz
feat: The functor of points of a scheme We construct the functor of points functor, and prove that it's full and faithful. --- - [ ] depends on: #11947 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebraic-geometry t-category-theory merge-conflict 210/0 Mathlib.lean,Mathlib/AlgebraicGeometry/FunctorOfPoints.lean,Mathlib/AlgebraicGeometry/OpenImmersion.lean 3 4 ['github-actions', 'grunweg', 'leanprover-community-mathlib4-bot'] nobody
294-85414
9 months ago
335-23470
11 months ago
0-1223
20 minutes
12418 rosborn
author:rosborn
style: replace preimage_val with ↓∩ notation --- This is a rough draft of what the new `↓∩` notation would look like within mathlib. I believe this is an improvement in clarity and would like to have `↓∩` as a standard notation (along with `''`, `⁻¹'`, `↑`, etc...). As `↓∩` is specialized for `Set`s, I have only changed `preimage_val` when the left-hand side of `↓∩` is a `Set`. The introduction of the `↓∩` notation to Data.Set.Image is temporary as it isn't possible to import Data.Set.Subset directly. If we want `↓∩` unscoped, where would be the best place to define it? An option is Data.Set.Defs, but the notation cannot be defined without additional imports as the file does not import `notation3`. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict 56/61 Mathlib/Analysis/InnerProductSpace/Projection.lean,Mathlib/Data/Set/Function.lean,Mathlib/Data/Set/Image.lean,Mathlib/Data/Set/Subset.lean,Mathlib/MeasureTheory/Constructions/Polish.lean,Mathlib/MeasureTheory/MeasurableSpace/Basic.lean,Mathlib/MeasureTheory/Measure/Restrict.lean,Mathlib/Order/UpperLower/Basic.lean,Mathlib/Topology/Bases.lean,Mathlib/Topology/Clopen.lean,Mathlib/Topology/Connected/Basic.lean,Mathlib/Topology/Connected/PathConnected.lean,Mathlib/Topology/Constructions.lean,Mathlib/Topology/ContinuousOn.lean,Mathlib/Topology/LocalAtTarget.lean,Mathlib/Topology/LocallyConstant/Basic.lean,Mathlib/Topology/Separation.lean,Mathlib/Topology/Sober.lean 18 3 ['grunweg', 'rosborn'] nobody
294-85313
9 months ago
335-23470
11 months ago
29-14218
29 days
9978 FR-vdash-bot
author:FR-vdash-bot
chore(FieldTheory/KummerExtension): move some lemmas earlier --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict awaiting-author
label:t-algebra$
197/177 Mathlib.lean,Mathlib/Data/Polynomial/FieldDivision.lean,Mathlib/FieldTheory/KummerExtension.lean,Mathlib/RingTheory/AdjoinRoot.lean,Mathlib/RingTheory/Polynomial/Irreducible.lean 5 5 ['alreadydone', 'grunweg', 'riccardobrasca'] nobody
294-85105
9 months ago
294-85105
9 months ago
8-83342
8 days
12429 adomani
author:adomani
feat: toND -- auto-generating natDegree This is an experiment to automatically translate theorems about `degree` to theorems about `natDegree`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra RFC t-meta merge-conflict awaiting-author
label:t-algebra$
167/132 Mathlib.lean,Mathlib/Algebra/Polynomial/Degree/Definitions.lean,Mathlib/Algebra/Polynomial/Degree/Lemmas.lean,Mathlib/Algebra/Polynomial/EraseLead.lean,Mathlib/Algebra/Polynomial/HasseDeriv.lean,Mathlib/Algebra/Polynomial/Inductions.lean,Mathlib/Algebra/Polynomial/Mirror.lean,Mathlib/Algebra/Polynomial/Reverse.lean,Mathlib/Tactic.lean,Mathlib/Tactic/ToNatDegree.lean,scripts/noshake.json 11 2 ['adomani', 'grunweg'] nobody
294-84416
9 months ago
294-84416
9 months ago
0-0
0 seconds
15823 eric-wieser
author:eric-wieser
Quotients of rings in model theory --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-logic merge-conflict 55/13 Mathlib/ModelTheory/Algebra/Ring/FreeCommRing.lean,Mathlib/ModelTheory/Syntax.lean 2 1 ['github-actions'] nobody
294-62979
9 months ago
294-62979
9 months ago
0-0
0 seconds
12178 joneugster
author:joneugster
feat(Data/Matrix/Basic): add notation for `m×n`-Matrices Introduce the notation `Mat[m,n][R]` for `Matrix (Fin m) (Fin n) R`. [Zulip thread](https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/Why.20does.20.60Matrix.2Erow.60.20use.20.20.60Unit.60.20instead.20of.20.60Fin.201.60.3F/near/427949223) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict
label:t-algebra$
139/135 Mathlib/Algebra/Lie/CartanMatrix.lean,Mathlib/Analysis/Complex/UpperHalfPlane/Basic.lean,Mathlib/Data/Matrix/Basic.lean,Mathlib/Data/Matrix/Notation.lean,Mathlib/Data/Matrix/Rank.lean,Mathlib/Data/Matrix/Reflection.lean,Mathlib/GroupTheory/Coxeter/Matrix.lean,Mathlib/LinearAlgebra/Matrix/Adjugate.lean,Mathlib/LinearAlgebra/Matrix/Charpoly/Coeff.lean,Mathlib/LinearAlgebra/Matrix/Determinant.lean,Mathlib/LinearAlgebra/Matrix/SpecialLinearGroup.lean,Mathlib/LinearAlgebra/Matrix/Trace.lean,Mathlib/LinearAlgebra/Matrix/Transvection.lean,Mathlib/LinearAlgebra/PID.lean,Mathlib/LinearAlgebra/Vandermonde.lean,Mathlib/NumberTheory/Modular.lean,Mathlib/NumberTheory/ModularForms/CongruenceSubgroups.lean,Mathlib/NumberTheory/ModularForms/SlashActions.lean,Mathlib/NumberTheory/ModularForms/SlashInvariantForms.lean,Mathlib/NumberTheory/RamificationInertia.lean,Mathlib/RingTheory/SimpleModule.lean,test/matrix.lean 22 9 ['YaelDillies', 'eric-wieser', 'grunweg', 'joneugster'] nobody
294-40103
9 months ago
294-44017
9 months ago
0-0
0 seconds
12751 Command-Master
author:Command-Master
feat: add lemmas for Nat/Bits, Nat/Bitwise and Nat/Size Remove `@[simp]` from `Nat.bit_false` and `Nat.bit_true`, as `bit0` and `bit1` are deprecated, and add some lemmas to `Bits`, `Bitwise` and `Size`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data new-contributor merge-conflict 66/7 Mathlib/Data/Nat/Bits.lean,Mathlib/Data/Nat/Bitwise.lean,Mathlib/Data/Nat/Multiplicity.lean,Mathlib/Data/Nat/Size.lean 4 26 ['Command-Master', 'Rida-Hamadani', 'Ruben-VandeVelde', 'YaelDillies', 'github-actions', 'jcommelin'] nobody
294-20067
9 months ago
299-36309
9 months ago
54-52408
54 days
9935 jstoobysmith
author:jstoobysmith
feat(AlgebraicTopology): add constructors for horns Added a function that given a simplicial set S and a set of n-1 simplexes satisfying certain conditions, creates a morphism in SSet from a n horn to a simplicial set S. Included also are a series of lemmas and definitions used in this construction. In particular I define a function that takes a m-simplex in a horn, and returns the smallest 'index' of face it factors through, and give a series of lemmas related to this. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra t-topology merge-conflict awaiting-author
label:t-algebra$
462/2 Mathlib/AlgebraicTopology/SimplicialSet.lean 1 15 ['YaelDillies', 'jcommelin', 'jstoobysmith', 'kim-em', 'linesthatinterlace'] nobody
294-19901
9 months ago
325-21226
10 months ago
14-58814
14 days
15448 urkud
author:urkud
chore(*): deprecate `Option.elim'` Use `Option.elim` instead. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) tech debt merge-conflict awaiting-author 54/50 Mathlib/Algebra/BigOperators/Option.lean,Mathlib/Algebra/MvPolynomial/Equiv.lean,Mathlib/Algebra/MvPolynomial/Variables.lean,Mathlib/Analysis/BoxIntegral/Partition/Additive.lean,Mathlib/Analysis/BoxIntegral/Partition/Basic.lean,Mathlib/Analysis/BoxIntegral/Partition/Split.lean,Mathlib/Analysis/Calculus/LagrangeMultipliers.lean,Mathlib/CategoryTheory/Category/PartialFun.lean,Mathlib/Computability/TMToPartrec.lean,Mathlib/Data/Option/Defs.lean,Mathlib/LinearAlgebra/Basis.lean,Mathlib/Logic/Embedding/Set.lean,Mathlib/Logic/Equiv/Basic.lean,Mathlib/MeasureTheory/OuterMeasure/Induced.lean,Mathlib/NumberTheory/Dioph.lean,Mathlib/Topology/Compactness/Paracompact.lean,Mathlib/Topology/LocallyFinite.lean 17 12 ['Ruben-VandeVelde', 'YaelDillies', 'github-actions', 'grunweg', 'urkud'] nobody
294-9120
9 months ago
294-84667
9 months ago
7-18420
7 days
10349 Shamrock-Frost
author:Shamrock-Frost
refactor(CategoryTheory/MorphismProperty) We make explicit some of the galois connections/closure operators in the existing MorphismProperty file, rewrite some proofs to take advantage of these structures, and change map/inverseImage by (1) swapping their argument order, for consistency with Set.range and Set.preimage and (2) making "map" perform the strict, evil map while "essMap" (previously called map) forms the closure of the image under isomorphisms. Finally we add `IsMultiplicative` instances for isos/epis/monos, with an eye towards constructing the wide subcategory on these classes of maps. --- - [x] depends on: #10347 - [ ] depends on: #10348 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory merge-conflict 474/318 Mathlib/CategoryTheory/Localization/Composition.lean,Mathlib/CategoryTheory/Localization/LocalizerMorphism.lean,Mathlib/CategoryTheory/MorphismProperty.lean,Mathlib/Data/Set/Lattice.lean,Mathlib/Order/Closure.lean,Mathlib/Order/Hom/Basic.lean,Mathlib/Order/Hom/CompleteLattice.lean,Mathlib/Order/RelIso/Basic.lean 8 1 ['leanprover-community-mathlib4-bot'] nobody
292-22350
9 months ago
335-23470
11 months ago
0-418
6 minutes
10350 Shamrock-Frost
author:Shamrock-Frost
feat(Data/Setoid): add the operations of taking the equivalence class of an element and of saturating a set wrt an equivalence relation I'm open to suggestions about changing the name "saturate", someone on zulip rightly pointed out this is a very overloaded term in math. That said, I think it's unlikely to cause confusion and that there's only one reasonable interpretation in the context of setoids. --- - [x] depends on: #10347 - [x] depends on: #10348 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data merge-conflict 169/3 Mathlib/Data/Setoid/Basic.lean,Mathlib/Data/Setoid/Partition.lean,Mathlib/Order/Closure.lean 3 1 ['leanprover-community-mathlib4-bot'] nobody
292-22341
9 months ago
299-36311
9 months ago
19-74514
19 days
13573 Shamrock-Frost
author:Shamrock-Frost
feat: add multivariate polynomial modules Add a type synonym for multivariate polynomials with coefficients in a module. --- Multivariate polynomials with module coefficients are sort of silly, but they sometimes show up in commutative algebra (eg in the definition of a quasi regular sequence). Writing this code involved a lot of copy and pasting from `PolynomialModule` and `MvPolynomial`. The API is definitely lacking at this stage but it's a start. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict awaiting-author
label:t-algebra$
691/6 Mathlib.lean,Mathlib/Algebra/MvPolynomial/Module/Basic.lean,Mathlib/Algebra/MvPolynomial/Module/MvAEval.lean,Mathlib/Algebra/Polynomial/Module/Basic.lean 4 9 ['Shamrock-Frost', 'erdOne', 'github-actions'] nobody
292-22321
9 months ago
298-32916
9 months ago
39-72739
39 days
6517 MohanadAhmed
author:MohanadAhmed
feat: discrete Fourier transform of a finite sequence # Discrete Fourier Transform (DFT) Matrix and DFT of a (finite) sequence This file defines the `dft` opertaion on a sequence (also a vecotr) and the DFT operation matrix ## Main definitions - `dft v`: given a sequence (v : (Fin n) → ℂ) we can transform it into a sequence (V : (Fin n) →ℂ) such that $$V [p] = ∑_{k = 0}^{N - 1} e^{-j*2πkp/n} v [k]$$ - `idft V` : given a sequence (V : (Fin n) → ℂ) we can transform it into a sequence (v : (Fin n) → ℂ) such that $$v [k] = \frac{1}{N}∑_{p = 0}^{n - 1} e^{j*2πkp/N} v [p]$$ - `dftMatrix n` : the dft matrix of dimensions $n \times n$ with the `k, p` entry equal to $$Wₙ[k, p] = e^{-j2πkp/n}$$ - `(dftMatrix n)⁻¹` : the idft matrix of dimensions $n \times n$ with the `k, p` entry equal to $$Wₙ[k, p] = (1/N) e^{j2πkp/n}$$ ## Main results - `dft v = (dftMatrix n) v` : the dft operation on a sequence is the same as the dft matrix applied to the vector - `idft V = (dftMatrix n)⁻¹ V` : the idft operation on a sequence is the same as the idft matrix applied to the vector - `dft (idft v) = dft ( idft v) = v` the dft and idft operations are inverses - `Wₙ = vandermonde (w)` : the dft matrix is vandermonde with `w` being the first row of the dft matrix - `circulant t = (dftMatrix n)⁻¹ ⬝ diagonal (dft t) ⬝ (dftMatrix n)` : a circulant matrix is diagonalizable by the dft and idft matrix pair. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict awaiting-author
label:t-algebra$
294/0 Mathlib.lean,Mathlib/LinearAlgebra/Matrix/DFT.lean 2 26 ['MohanadAhmed', 'ericrbg'] nobody
292-22159
9 months ago
371-11749
1 year ago
65-20427
65 days
13155 alreadydone
author:alreadydone
feat(NumberTheory/EllipticDivisibilitySequence): show elliptic relations follow from even-odd recursion This PR is centered around the (generalized) elliptic relations (`rel₄`) $E(a,b,c,d): W_{a+b}W_{a-b}W_{c+d}W_{c-d}=W_{a+c}W_{a-c}W_{b+d}W_{b-d}-W_{a+d}W_{a-d}W_{b+c}W_{b-c}$. For an integer-indexed sequence W valued in a commutative ring, the relation makes sense only when a,b,c,d are all integers or all half integers. For convenience of formalization, we instead consider integers a,b,c,d of the same parity and divide all subscripts by 2. We extract the subexpression $W_{(a+b)/2}W_{(a-b)/2}$ (which appear six times) as `addMulSub W a b`. The collection of all $E(a,b,c,d)$ is equivalent to Stange's axiom for elliptic nets (`net`), and the literature (e.g. Silverman) commonly consider only the three-index special case $E(m,n,r,0)$ (`Rel₃`). Important special cases of these relations are (i) $E(m+1,m,1,0): W_{2m+1}W_1^3=W_{m+2}W_m^3-W_{m+1}^3 W_{m-1}$ (`oddRec`) and (ii) $E(m+1,m-1,1,0): W_{2m}W_2 W_1^2=W_m(W_{m+2}W_{m-1}^2-W_{m-2}W_{m+1}^2)$ (`evenRec`), which suffice to uniquely specify $W$ on all positive integers recursively from four initial values $W_1, W_2, W_3, W_4$ (`IsEllSequence.ext`, if $W_1 W_2$ is not a zero divisor). In the usual setting where $W_1=1$ and $W_2\mid W_4$, there does exist a sequence (`normEDS`) satisfying (i) and (ii) given initial values $W_2, W_3$ and $W_4/W_2$. It turns out the same non-zerodivisor condition also guarantees that W is an odd function with $W_0=0$, which naturally extends W to all integers. The main result of this PR (`rel₄_of_oddRec_evenRec`, `IsEllSequence.of_oddRec_evenRec`) is a purely algebraic proof that the sequence W defined by the single-parameter elliptic relations (i) and (ii) implies all $E(a,b,c,d)$, based on my original argument first published on [Math.SE](https://math.stackexchange.com/a/4903422/12932). It's based on the observation that a nonzerodivisor-multiple of $E(a,b,c,d)$ can be expressed as a linear combination of various $E(a,b,c_\min,d_\min)$ with the two smallest indices fixed at their minimal possible values, which can be transformed (`transf`) to an elliptic relation with smaller `a` (which can be assumed to hold by induction), unless they are of the form (i) or (ii) which hold by assumption. For this argument it's necessary to assume `a > b > c > d ≥ 0` (see `StrictAnti₄` and `Rel₄OfValid`), but it's easy to extend to arbitrary a,b,c,d by symmetry properties of `rel₄` under negation and permutations of indices. In the subsequent PR #13057, we show all normalized EDSs (`normEDS`), defined using the even-odd recursion (i)-(ii), are elliptic (i.e. satisfy the elliptic relations) divisibility sequences. This PR doesn't directly apply because a normEDS doesn't always satisfy the nonzerodivisor condition, but they are specializations of the universal normEDS, which does satisfy the condition. The technique of reducing to the universal case will be applied many times, and relies on the naturality (`map`) lemmas. We also change the `ℕ` in the definition `IsDivSequence` to `ℤ` which is more natural given that W is a `ℤ`-indexed sequence. --- - [x] depends on: #13153 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-number-theory merge-conflict awaiting-author
label:t-algebra$
565/12 Mathlib/NumberTheory/EllipticDivisibilitySequence.lean 1 55 ['Multramate', 'alreadydone', 'github-actions', 'grunweg', 'leanprover-community-mathlib4-bot'] nobody
286-35763
9 months ago
286-35763
9 months ago
26-39367
26 days
15600 adomani
author:adomani
feat: lint also `let` vs `have` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-linter merge-conflict WIP 77/26 Mathlib/Tactic/Linter/HaveLetLinter.lean,test/HaveLetLinter.lean 2 1 ['github-actions'] nobody
285-4039
9 months ago
285-4039
9 months ago
0-8
8 seconds
13970 adomani
author:adomani
feat: a linter to flag unnecessary uses of `nolint simpNF` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-linter merge-conflict awaiting-author 230/0 Mathlib.lean,Mathlib/Analysis/CStarAlgebra/Basic.lean,Mathlib/Analysis/Quaternion.lean,Mathlib/CategoryTheory/Comma/Arrow.lean,Mathlib/CategoryTheory/Monoidal/End.lean,Mathlib/Data/NNRat/Defs.lean,Mathlib/Data/Rat/Defs.lean,Mathlib/LinearAlgebra/CliffordAlgebra/Even.lean,Mathlib/LinearAlgebra/CliffordAlgebra/EvenEquiv.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter.lean,Mathlib/Tactic/Linter/UnnecessarySyntax.lean,test/UnnecessarySyntax.lean 13 4 ['adomani', 'github-actions', 'grunweg', 'leanprover-bot'] nobody
283-27253
9 months ago
283-27254
9 months ago
0-0
0 seconds
14923 Multramate
author:Multramate
feat(AlgebraicGeometry/EllipticCurve/Jacobian): add equivalences between points and explicit WithZero types --- - [ ] depends on: #14627 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebraic-geometry t-number-theory merge-conflict blocked-by-other-PR 262/66 Mathlib/AlgebraicGeometry/EllipticCurve/Affine.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Group.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Jacobian.lean,scripts/style-exceptions.txt 4 2 ['github-actions', 'leanprover-community-mathlib4-bot'] nobody
283-27126
9 months ago
283-27126
9 months ago
0-0
0 seconds
15162 adomani
author:adomani
feat: checkAsSorry linter A very preliminary version of the `checkAsSorry` linter. It flags declarations whose type is not equal to the 'asSorry'ed one. [Zulip discussion](https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/Running.20Mathlib.20under.20.60set_option.20debug.2EbyAsSorry.60) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-linter merge-conflict 119/0 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter/CheckAsSorry.lean,test/CheckAsSorry.lean 4 1 ['github-actions'] nobody
283-26241
9 months ago
283-26241
9 months ago
0-0
0 seconds
14266 dagurtomas
author:dagurtomas
feat(AlgebraicGeometry): define a pretopology from a RingHomProperty --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) workshop-AIM-AG-2024 t-algebraic-geometry merge-conflict please-adopt WIP 101/0 Mathlib/AlgebraicGeometry/Morphisms/RingHomProperties.lean,Mathlib/CategoryTheory/Sites/MorphismProperty.lean,Mathlib/CategoryTheory/Sites/Pretopology.lean 3 1 ['github-actions'] nobody
280-36421
9 months ago
280-36421
9 months ago
0-0
0 seconds
14046 adomani
author:adomani
test: diff of declarations in lean --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP 231/2 .github/workflows/bors.yml,.github/workflows/build.yml,.github/workflows/build.yml.in,.github/workflows/build_fork.yml,.github/workflows/mk_build_yml.sh,Mathlib/Tactic/Eval.lean,scripts/decls_diff_hybrid.sh,scripts/list_decls.lean 8 2 ['github-actions'] nobody
279-19755
9 months ago
279-19755
9 months ago
0-0
0 seconds
14038 adomani
author:adomani
test/decl diff in lean dev --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP 231/2 .github/workflows/bors.yml,.github/workflows/build.yml,.github/workflows/build.yml.in,.github/workflows/build_fork.yml,.github/workflows/mk_build_yml.sh,Mathlib/Tactic/Eval.lean,scripts/decls_diff_hybrid.sh,scripts/list_decls.lean 8 3 ['github-actions'] nobody
279-19755
9 months ago
279-19755
9 months ago
0-0
0 seconds
12107 yuma-mizuno
author:yuma-mizuno
feat(Mathlib/Tactic/Widget/StringDiagram): support 2-morphisms in bicategories --- - [x] depends on: #11080 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory t-meta merge-conflict 1158/0 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/CategoryTheory/Coherence.lean,Mathlib/Tactic/Widget/StringDiagram.lean,scripts/noshake.json,test/StringDiagram.lean,widget/src/penrose/monoidal.dsl,widget/src/penrose/monoidal.sty 8 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
274-14499
9 months ago
274-14502
9 months ago
0-0
0 seconds
15925 yuma-mizuno
author:yuma-mizuno
feat(CategoryTheory/Monoida): proof producing coherence tactic --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory t-meta merge-conflict 5018/265 Mathlib.lean,Mathlib/CategoryTheory/Bicategory/Adjunction.lean,Mathlib/CategoryTheory/Bicategory/Kan/Adjunction.lean,Mathlib/CategoryTheory/Monoidal/Braided/Basic.lean,Mathlib/CategoryTheory/Monoidal/CoherenceLemmas.lean,Mathlib/CategoryTheory/Monoidal/Opposite.lean,Mathlib/CategoryTheory/Monoidal/Rigid/Basic.lean,Mathlib/CategoryTheory/Monoidal/Rigid/Braided.lean,Mathlib/Tactic.lean,Mathlib/Tactic/CategoryTheory/BicategoricalComp.lean,Mathlib/Tactic/CategoryTheory/Bicategory/Normalize.lean,Mathlib/Tactic/CategoryTheory/Bicategory/PureCoherence.lean,Mathlib/Tactic/CategoryTheory/Coherence.lean,Mathlib/Tactic/CategoryTheory/Coherence/Basic.lean,Mathlib/Tactic/CategoryTheory/Coherence/Datatypes.lean,Mathlib/Tactic/CategoryTheory/Coherence/Normalize.lean,Mathlib/Tactic/CategoryTheory/Coherence/PureCoherence.lean,Mathlib/Tactic/CategoryTheory/CoherenceNew.lean,Mathlib/Tactic/CategoryTheory/Monoidal.lean,Mathlib/Tactic/CategoryTheory/Monoidal/Basic.lean,Mathlib/Tactic/CategoryTheory/Monoidal/Datatypes.lean,Mathlib/Tactic/CategoryTheory/Monoidal/Normalize.lean,Mathlib/Tactic/CategoryTheory/Monoidal/PureCoherence.lean,Mathlib/Tactic/CategoryTheory/MonoidalComp.lean,Mathlib/Tactic/Widget/StringDiagram.lean,lake-manifest.json,scripts/noshake.json,test/CategoryTheory/Bicategory.lean,test/CategoryTheory/Coherence.lean,test/CategoryTheory/CoherenceNew.lean,test/CategoryTheory/Monoidal.lean,test/CategoryTheory/Monoidal/Basic.lean,test/CategoryTheory/Monoidal/Normalize.lean,test/CategoryTheory/MonoidalComp.lean,test/StringDiagram.lean 35 n/a ['github-actions'] nobody
273-61036
9 months ago
unknown
unknown
7861 shuxuezhuyi
author:shuxuezhuyi
feat(Geometry/Hyperbolic/UpperHalfPlane): instance IsometricSMul PSL(2, ℝ) ℍ --- - [ ] depends on: #7835 - [ ] depends on: #7791 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-euclidean-geometry merge-conflict blocked-by-other-PR 98/0 Mathlib.lean,Mathlib/Geometry/Hyperbolic/UpperHalfPlane/Basic.lean,Mathlib/LinearAlgebra/Matrix/ProjectiveSpecialLinearGroup.lean 3 1 ['leanprover-community-mathlib4-bot'] nobody
273-42096
9 months ago
273-42096
9 months ago
0-0
0 seconds
6475 joneugster
author:joneugster
refactor(LinearAlgebra/Span): replace ∙ with • as notation for `span R {x}` Change the notation for `Submodule.span R {x}` from `R ∙ x` to the bullet `R • x`, which is also used for scalar multiplication. --- (this was an experiment originating from a [Zulip discussion](https://leanprover.zulipchat.com/#narrow/stream/270676-lean4/topic/.2E.C2.B7.E2.AC.9D.20.5Brant.5D), I don't have a clear opinion if this is actually a desired thing to do...) Generally this works and Lean seems to do fine figuring out the difference between `r • x` and `R • x` (The former is scalar multiplication in an `R`-module `M`, the latter is the `Submodule R M` generated by `x`). Encountered a few regressions that should be considered (the first two might be also bugs that could be looked at independently): 1. `(· • ·)`, and general simple function syntax, does not work as notation for `HSMul.hSMul` anymore. For this reason, I introduced the notation `scoped` to minimise the effect of this. Now it's only a problem if you `open Span`. Note that `fun x₁ x₂ ↦ x₁ • x₂` works flawlessly all the time. 4. `change` and `convert` have troubles to deal with the two competing notations. `have := _; convert this` works. 5. `R • x - y` is not valid anymore and needs parentheses: `R • (x - y)`. I do think this actually helps readability, so I don't mind. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra RFC merge-conflict
label:t-algebra$
323/240 Mathlib/Algebra/Algebra/Operations.lean,Mathlib/Algebra/Algebra/Subalgebra/Basic.lean,Mathlib/Algebra/Lie/Engel.lean,Mathlib/Algebra/Lie/Normalizer.lean,Mathlib/Algebra/Module/PID.lean,Mathlib/Algebra/Module/Torsion.lean,Mathlib/Analysis/InnerProductSpace/Basic.lean,Mathlib/Analysis/InnerProductSpace/GramSchmidtOrtho.lean,Mathlib/Analysis/InnerProductSpace/Orthogonal.lean,Mathlib/Analysis/InnerProductSpace/PiL2.lean,Mathlib/Analysis/InnerProductSpace/Projection.lean,Mathlib/Analysis/InnerProductSpace/TwoDim.lean,Mathlib/Analysis/NormedSpace/ContinuousLinearMap.lean,Mathlib/Analysis/NormedSpace/HahnBanach/Extension.lean,Mathlib/Analysis/NormedSpace/OperatorNorm.lean,Mathlib/Data/ZMod/Quotient.lean,Mathlib/Geometry/Euclidean/Angle/Oriented/Basic.lean,Mathlib/Geometry/Euclidean/Inversion/Calculus.lean,Mathlib/Geometry/Euclidean/MongePoint.lean,Mathlib/Geometry/Euclidean/PerpBisector.lean,Mathlib/Geometry/Euclidean/Sphere/SecondInter.lean,Mathlib/Geometry/Manifold/Instances/Sphere.lean,Mathlib/LinearAlgebra/AffineSpace/AffineSubspace.lean,Mathlib/LinearAlgebra/AffineSpace/FiniteDimensional.lean,Mathlib/LinearAlgebra/BilinearForm.lean,Mathlib/LinearAlgebra/DFinsupp.lean,Mathlib/LinearAlgebra/Dimension.lean,Mathlib/LinearAlgebra/FiniteDimensional.lean,Mathlib/LinearAlgebra/LinearIndependent.lean,Mathlib/LinearAlgebra/LinearPMap.lean,Mathlib/LinearAlgebra/ProjectiveSpace/Basic.lean,Mathlib/LinearAlgebra/QuadraticForm/Basic.lean,Mathlib/LinearAlgebra/Quotient.lean,Mathlib/LinearAlgebra/SesquilinearForm.lean,Mathlib/LinearAlgebra/Span.lean,Mathlib/MeasureTheory/Integral/Periodic.lean,Mathlib/RingTheory/Coprime/Ideal.lean,Mathlib/RingTheory/Finiteness.lean,Mathlib/RingTheory/Ideal/AssociatedPrime.lean,Mathlib/RingTheory/Ideal/IdempotentFG.lean,Mathlib/RingTheory/Noetherian.lean,Mathlib/Topology/Instances/AddCircle.lean 42 3 ['eric-wieser', 'joneugster', 'leanprover-bot'] nobody
272-39392
8 months ago
272-39392
8 months ago
0-0
0 seconds
7545 shuxuezhuyi
author:shuxuezhuyi
feat: APIs of `Function.extend f g e'` when `f` is injective We characterizes `range g`, `Injective g`, `Surjective g` and `Bijective g` in terms of `extend f g e'`.​ --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-logic merge-conflict awaiting-author 50/0 Mathlib.lean,Mathlib/Logic/Function/ApiForExtend.lean 2 1 ['fpvandoorn'] nobody
271-54928
8 months ago
271-54928
8 months ago
32-30254
32 days
10765 Vierkantor
author:Vierkantor
feat(Tactic): `ring` modulo a given characteristic This PR extends the `ring` tactic with a new config argument `char` which will try to reduce all constant terms modulo the given characteristic. This allows `ring` to prove e.g. `(x + y)^3 = x^3 + y^3` in characteristic 3. This is a simpler and faster way to do so than what we had before: `repeat { ring; reduce_mod_char }` becomes `ring (config := { char := 3 })`. The first step is to split off the required `CharP` definitions, since `Mathlib.Algebra.CharP.Basic` already requires the `ring` tactic. To perform the reduction modulo the given characteristic, I implemented `reduceCast` which reduces a raw integer, and wrapped it in `reduceResult` that takes a `NormNum.Result` for easy use. We need to pass through quite a few parameters into `reduceResult` so maybe it's worth defining a structure, or reusing `Cache` for this. Then it's basically a case of replacing every place where `ring` constructs a numeral with a call to `reduceResult`. Limitations: * `ring` doesn't attempt to detect the characteristic by itself, you need to pass it in explicitly. Trying to infer a `CharP` instance at each point sounds quite expensive. * Since the support for `%` in `NormNum` only exists for integers, I implemented the reduction only when a `Ring` instance is available. It is still sound in the semiring case, just not complete. * We could optimize exponentiation in the specific case where the characteristic `p` is a prime that divides the exponent `n`: `(x + y)^n = x^n + y^n`. I'll leave that to future work. --- - [x] depends on: #12907 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta merge-conflict awaiting-author help-wanted 275/108 Mathlib/RingTheory/MvPolynomial/Basic.lean,Mathlib/Tactic/Polyrith.lean,Mathlib/Tactic/Ring/Basic.lean,Mathlib/Tactic/Ring/RingNF.lean,test/ring_mod_char.lean 5 7 ['Vierkantor', 'YaelDillies', 'github-actions', 'joneugster', 'leanprover-community-mathlib4-bot'] joneugster
assignee:joneugster
271-24622
8 months ago
271-24622
8 months ago
28-28613
28 days
12632 urkud
author:urkud
feat(List/OffDiag): new file --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data merge-conflict awaiting-author 184/3 Mathlib.lean,Mathlib/Data/List/Basic.lean,Mathlib/Data/List/Enum.lean,Mathlib/Data/List/EraseIdx.lean,Mathlib/Data/List/OffDiag.lean 5 3 ['eric-wieser', 'github-actions', 'urkud'] nobody
268-25743
8 months ago
268-25743
8 months ago
0-0
0 seconds
16658 adomani
author:adomani
add tips file --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) test-ci merge-conflict awaiting-author WIP 51/508 .github/build.in.yml,.github/workflows/bors.yml,.github/workflows/build.yml,.github/workflows/build_fork.yml,scripts/Tips.lean 5 1 ['github-actions'] nobody
267-83861
8 months ago
267-83861
8 months ago
0-0
0 seconds
14078 Ruben-VandeVelde
author:Ruben-VandeVelde
feat(CI): continue after mk_all fails --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) CI merge-conflict awaiting-author 43/0 .github/workflows/bors.yml,.github/workflows/build.yml,.github/workflows/build.yml.in,.github/workflows/build_fork.yml,Mathlib/Data/Nat/Test.lean 5 2 ['bryangingechen', 'github-actions'] nobody
267-64161
8 months ago
267-64161
8 months ago
0-0
0 seconds
11800 JADekker
author:JADekker
feat : Define KappaLindelöf spaces Define KappaLindelöf spaces by following the first one-third of the API for Lindelöf spaces. The remainder will be added in a future PR. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-zulip t-topology merge-conflict please-adopt 301/2 Mathlib.lean,Mathlib/Topology/Compactness/KappaLindelof.lean,Mathlib/Topology/Compactness/Lindelof.lean 3 38 ['ADedecker', 'JADekker', 'PatrickMassot', 'StevenClontz', 'adomani', 'github-actions', 'grunweg', 'kim-em', 'urkud'] nobody
266-54938
8 months ago
266-76913
8 months ago
119-10687
119 days
12087 JADekker
author:JADekker
feat : complete API for K-Lindelöf spaces --- - [ ] depends on: #11800 (which is now awaiting a design decision) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology merge-conflict please-adopt blocked-by-other-PR 789/17 Mathlib.lean,Mathlib/Order/Filter/CardinalInter.lean,Mathlib/Topology/Compactness/KLindelof.lean,Mathlib/Topology/Compactness/Lindelof.lean 4 2 ['github-actions', 'leanprover-community-mathlib4-bot'] nobody
266-54680
8 months ago
266-54680
8 months ago
1-72084
1 day
11283 hmonroe
author:hmonroe
feat(ModelTheory/Satisfiability): define theory with independent sentence --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-logic merge-conflict WIP 8/0 Mathlib/ModelTheory/Satisfiability.lean 1 2 ['fpvandoorn', 'hmonroe'] nobody
265-34715
8 months ago
265-34715
8 months ago
3-5240
3 days
16914 siddhartha-gadgil
author:siddhartha-gadgil
Loogle syntax with non-reserved This is PR mainly to test that loogle syntax does not break stuff downstream --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP 4/4 lake-manifest.json,lakefile.lean 2 1 ['github-actions'] nobody
263-23324
8 months ago
263-23324
8 months ago
0-14835
4 hours
10075 dupuisf
author:dupuisf
refactor: generalize `MonoidHom.ker` and `MonoidHom.range` to `MonoidHomClass` With this refactor, `MonoidHom.ker` and `MonoidHom.range` will be defined for any `MonoidHomClass` type, not just `MonoidHom`s. This brings the design in line with `LinearMap.ker`/`range` and `MonoidHom.mker`/`mrange`. `Subgroup.map`/`comap` are also generalized. As with those previous refactors, the main drawback is the loss of dot notation in many cases. Other than that, the impact is fairly minor given that this is happening is rather basic files. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict awaiting-author
label:t-algebra$
464/389 Mathlib/Algebra/Category/GroupCat/Abelian.lean,Mathlib/Algebra/Category/GroupCat/Basic.lean,Mathlib/Algebra/Category/GroupCat/Colimits.lean,Mathlib/Algebra/Category/GroupCat/EpiMono.lean,Mathlib/Algebra/Category/GroupCat/Images.lean,Mathlib/Algebra/Category/GroupCat/Kernels.lean,Mathlib/Algebra/Category/GroupCat/Limits.lean,Mathlib/Algebra/Homology/ShortComplex/Ab.lean,Mathlib/Analysis/Normed/Group/Basic.lean,Mathlib/Analysis/Normed/Group/Hom.lean,Mathlib/Data/ZMod/Basic.lean,Mathlib/Data/ZMod/Quotient.lean,Mathlib/FieldTheory/PolynomialGaloisGroup.lean,Mathlib/GroupTheory/Abelianization.lean,Mathlib/GroupTheory/CoprodI.lean,Mathlib/GroupTheory/Coset.lean,Mathlib/GroupTheory/Finiteness.lean,Mathlib/GroupTheory/FreeGroup/Basic.lean,Mathlib/GroupTheory/GroupAction/Quotient.lean,Mathlib/GroupTheory/HNNExtension.lean,Mathlib/GroupTheory/Index.lean,Mathlib/GroupTheory/Nilpotent.lean,Mathlib/GroupTheory/NoncommPiCoprod.lean,Mathlib/GroupTheory/PGroup.lean,Mathlib/GroupTheory/Perm/Sign.lean,Mathlib/GroupTheory/Perm/Subgroup.lean,Mathlib/GroupTheory/PushoutI.lean,Mathlib/GroupTheory/QuotientGroup.lean,Mathlib/GroupTheory/SchurZassenhaus.lean,Mathlib/GroupTheory/SemidirectProduct.lean,Mathlib/GroupTheory/Solvable.lean,Mathlib/GroupTheory/SpecificGroups/Alternating.lean,Mathlib/GroupTheory/SpecificGroups/Cyclic.lean,Mathlib/GroupTheory/Subgroup/Basic.lean,Mathlib/GroupTheory/Subgroup/Finite.lean,Mathlib/GroupTheory/Subgroup/Saturated.lean,Mathlib/GroupTheory/Subgroup/ZPowers.lean,Mathlib/GroupTheory/Sylow.lean,Mathlib/GroupTheory/Torsion.lean,Mathlib/GroupTheory/Transfer.lean,Mathlib/LinearAlgebra/Alternating/DomCoprod.lean,Mathlib/LinearAlgebra/Basic.lean,Mathlib/LinearAlgebra/Matrix/Determinant.lean,Mathlib/MeasureTheory/Function/LpSpace.lean,Mathlib/NumberTheory/ModularForms/CongruenceSubgroups.lean,Mathlib/RingTheory/ClassGroup.lean,Mathlib/RingTheory/DedekindDomain/SelmerGroup.lean,Mathlib/RingTheory/Valuation/ValuationSubring.lean,Mathlib/Topology/Algebra/OpenSubgroup.lean,Mathlib/Topology/Algebra/UniformGroup.lean,Mathlib/Topology/Instances/AddCircle.lean 51 2 ['dupuisf', 'urkud'] nobody
263-21213
8 months ago
263-52478
8 months ago
8-14499
8 days
10991 thorimur
author:thorimur
feat: `tfae` block tactic This PR introduces `tfae` block tactic syntax: ```lean tfae 1 → 2 := /- proof of `P₁ → P₂` -/ 2 → 3 := /- proof of `P₂ → P₃` -/ 3 → 1 := /- proof of `P₃ → P₁` -/ ``` Like the recent change to `tfae_have`, this syntax also supports all sorts of matching that `have` itself supports: ```lean tfae 2 → 3 | h₂ => /- proof of `P₃` -/ 3 → 1 -- given `P₁ := ∀(a : A), (b : B), (c : C), X`: | h₃, a, b, c => /- proof of `X` -/ ⟨h_mp, h_mpr⟩ : 1 ↔ 2 := /- proof of `P₁ ↔ P₂`; puts `h_mp : P₁ → P₂`, `h_mpr : P₂ → P₁` in the lctx -/ ``` This initial implementation is currently very simple, and relies on `tfae_have` and `tfae_finish`. Although we intend to migrate away from that syntax, this PR does not remove support for it or deprecate `tfae_have`/`tfae_finish` in any way; migration (but not deprecation) is done in #11003. --- - [ ] depends on: #10653 - [x] depends on: #10994 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta merge-conflict modifies-tactic-syntax WIP 392/124 Mathlib/Tactic/TFAE.lean,scripts/noshake.json,test/tfae.lean 3 3 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
262-46978
8 months ago
262-46978
8 months ago
0-0
0 seconds
16464 Parcly-Taxel
author:Parcly-Taxel
chore: deprecate `Nat.(case_)strong_induction_on` …in favour of the now-renamed `Nat.(case)strongInductionOn` in core. tech debt merge-conflict 54/56 Archive/Imo/Imo1981Q3.lean,Mathlib/Algebra/ContinuedFractions/Computation/Approximations.lean,Mathlib/Algebra/ContinuedFractions/Computation/TerminatesIffRat.lean,Mathlib/Algebra/ContinuedFractions/ConvergentsEquiv.lean,Mathlib/Algebra/Polynomial/Derivative.lean,Mathlib/Algebra/Polynomial/Lifts.lean,Mathlib/Analysis/Analytic/Basic.lean,Mathlib/Analysis/Calculus/ContDiff/Bounds.lean,Mathlib/Analysis/Hofer.lean,Mathlib/Analysis/SpecificLimits/Normed.lean,Mathlib/Combinatorics/Derangements/Finite.lean,Mathlib/Combinatorics/Enumerative/Catalan.lean,Mathlib/Combinatorics/Hall/Finite.lean,Mathlib/Combinatorics/SetFamily/AhlswedeZhang.lean,Mathlib/Computability/Primrec.lean,Mathlib/Data/Fintype/Basic.lean,Mathlib/Data/Fintype/Card.lean,Mathlib/Data/Nat/Choose/Central.lean,Mathlib/Data/Nat/Defs.lean,Mathlib/Data/Nat/Digits.lean,Mathlib/Data/Nat/Log.lean,Mathlib/FieldTheory/Separable.lean,Mathlib/LinearAlgebra/Eigenspace/Triangularizable.lean,Mathlib/LinearAlgebra/Multilinear/Basic.lean,Mathlib/NumberTheory/BernoulliPolynomials.lean,Mathlib/NumberTheory/DiophantineApproximation.lean,Mathlib/NumberTheory/Pell.lean,Mathlib/NumberTheory/Primorial.lean,Mathlib/Order/Fin/Basic.lean,Mathlib/RingTheory/Adjoin/PowerBasis.lean,Mathlib/RingTheory/LittleWedderburn.lean,Mathlib/RingTheory/Polynomial/Basic.lean,Mathlib/RingTheory/Polynomial/Cyclotomic/Basic.lean,Mathlib/RingTheory/Polynomial/Cyclotomic/Eval.lean,Mathlib/RingTheory/Polynomial/Eisenstein/IsIntegral.lean,Mathlib/RingTheory/Polynomial/Nilpotent.lean,Mathlib/RingTheory/PowerSeries/Basic.lean,Mathlib/RingTheory/QuotientNilpotent.lean,Mathlib/RingTheory/WittVector/Defs.lean,Mathlib/RingTheory/WittVector/Frobenius.lean,Mathlib/RingTheory/WittVector/StructurePolynomial.lean,Mathlib/SetTheory/Surreal/Dyadic.lean,Mathlib/Topology/Metrizable/Uniformity.lean 43 13 ['Parcly-Taxel', 'b-mehta', 'github-actions', 'jcommelin'] nobody
262-8623
8 months ago
262-8623
8 months ago
8-1989
8 days
13782 alreadydone
author:alreadydone
feat(EllipticCurve): ZSMul formula in terms of division polynomials The formula $[n]P = (\phi_n(x,y) : \omega_n(x,y) : \psi_n(x,y))$ in Jacobian coordinates for $P=(x,y)$ a nonsingular point on a Weierstrass/elliptic curve. --- - [x] depends on: #12883 - [x] depends on: #13399 - [ ] depends on: #13057 - [ ] depends on: #13155 - [x] depends on: #13845 - [x] depends on: #13846 - [ ] depends on: #13847 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-algebraic-geometry t-number-theory merge-conflict blocked-by-other-PR
label:t-algebra$
2462/232 Mathlib.lean,Mathlib/Algebra/MvPolynomial/PDeriv.lean,Mathlib/Algebra/Polynomial/Bivariate.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Affine.lean,Mathlib/AlgebraicGeometry/EllipticCurve/DivisionPolynomial/Basic.lean,Mathlib/AlgebraicGeometry/EllipticCurve/DivisionPolynomial/ZSMul.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Group.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Jacobian.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Universal.lean,Mathlib/NumberTheory/EllipticDivisibilitySequence.lean 10 n/a ['Multramate', 'alreadydone', 'github-actions', 'leanprover-community-mathlib4-bot'] nobody
260-72689
8 months ago
unknown
unknown
8118 iwilare
author:iwilare
feat(CategoryTheory): add dinatural transformations A starting point to define [dinatural transformations](https://ncatlab.org/nlab/show/dinatural+transformation). This is my first PR so style comments and improvements are very welcome! --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory merge-conflict awaiting-author 147/7 Mathlib.lean,Mathlib/CategoryTheory/DinatTrans.lean,Mathlib/CategoryTheory/Functor/Category.lean,Mathlib/CategoryTheory/Products/Bifunctor.lean 4 49 ['Shamrock-Frost', 'github-actions', 'iwilare', 'joelriou'] Shamrock-Frost
assignee:Shamrock-Frost
258-45610
8 months ago
258-45611
8 months ago
21-9462
21 days
10006 jstoobysmith
author:jstoobysmith
feat(AlgebraicTopology): homotopy in quasicategories Defined a homotopy between two 1-simplicies in a quasicategories, and proved the property of being homotopic forms an equivalence relation. --- - [ ] depends on: #9935 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-category-theory merge-conflict awaiting-author blocked-by-other-PR 898/1 Mathlib.lean,Mathlib/AlgebraicTopology/Homotopy.lean,Mathlib/AlgebraicTopology/SimplexCategory.lean,Mathlib/AlgebraicTopology/SimplicialSet.lean 4 3 ['joelriou', 'leanprover-community-mathlib4-bot'] nobody
258-45486
8 months ago
258-45486
8 months ago
0-0
0 seconds
14242 js2357
author:js2357
feat: Prove equivalence of `isDedekindDomain` and `isDedekindDomainDvr` Prove that `isDedekindDomainDvr` is equivalent to both `isDedekindDomain` and `isDedekindDomainInv`. Specifically, prove `isDedekindDomainDvr A → isDedekindDomainInv A`, because `isDedekindDomain A → isDedekindDomainDvr A` and `IsDedekindDomain A ↔ IsDedekindDomainInv A` are already in Mathlib. - [x] depends on: #14099 - [x] depends on: #14216 - [ ] depends on: #14237 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra merge-conflict blocked-by-other-PR
label:t-algebra$
269/1 Mathlib.lean,Mathlib/RingTheory/DedekindDomain/Dvr.lean,Mathlib/RingTheory/FractionalIdeal/LocalizedAtPrime.lean,Mathlib/RingTheory/Localization/Basic.lean 4 2 ['github-actions', 'leanprover-community-mathlib4-bot'] nobody
258-5961
8 months ago
258-5961
8 months ago
0-0
0 seconds
17110 FR-vdash-bot
author:FR-vdash-bot
chore: deprecate some lemmas about equality These lemmas were upstreamed to Batteries in https://github.com/leanprover-community/batteries/pull/465. --- - [ ] depends on: https://github.com/leanprover-community/batteries/pull/957 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-batt-PR merge-conflict 20/16 Mathlib/Combinatorics/SimpleGraph/Walk.lean,Mathlib/Data/Nat/Bitwise.lean,Mathlib/Logic/Basic.lean,Mathlib/Logic/Equiv/Basic.lean,Mathlib/Tactic/CC/Addition.lean,lake-manifest.json 6 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
254-8397
8 months ago
254-8399
8 months ago
0-0
0 seconds
17171 FR-vdash-bot
author:FR-vdash-bot
test extends carrier and property --- We need https://github.com/leanprover/lean4/issues/2666 ... [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict 433/309 Mathlib/Algebra/Algebra/NonUnitalSubalgebra.lean,Mathlib/Algebra/Algebra/Subalgebra/Basic.lean,Mathlib/Algebra/Algebra/Subalgebra/Directed.lean,Mathlib/Algebra/DirectSum/Decomposition.lean,Mathlib/Algebra/Field/Subfield.lean,Mathlib/Algebra/Group/Subgroup/Basic.lean,Mathlib/Algebra/Group/Subgroup/MulOpposite.lean,Mathlib/Algebra/Group/Submonoid/Basic.lean,Mathlib/Algebra/Group/Submonoid/MulOpposite.lean,Mathlib/Algebra/Group/Submonoid/Pointwise.lean,Mathlib/Algebra/Group/Submonoid/Units.lean,Mathlib/Algebra/Group/Subsemigroup/Basic.lean,Mathlib/Algebra/Group/Subsemigroup/Operations.lean,Mathlib/Algebra/Module/Submodule/Basic.lean,Mathlib/Algebra/Module/Submodule/Lattice.lean,Mathlib/Algebra/Module/Submodule/Map.lean,Mathlib/Algebra/Module/Submodule/Pointwise.lean,Mathlib/Algebra/Ring/Subring/Basic.lean,Mathlib/Algebra/Ring/Subsemiring/Basic.lean,Mathlib/Algebra/Ring/Subsemiring/MulOpposite.lean,Mathlib/Algebra/Ring/Subsemiring/Order.lean,Mathlib/Algebra/Star/Subalgebra.lean,Mathlib/Algebra/Star/Subsemiring.lean,Mathlib/Data/Complex/Module.lean,Mathlib/Data/SetLike/Basic.lean,Mathlib/Deprecated/Subfield.lean,Mathlib/Deprecated/Subgroup.lean,Mathlib/Deprecated/Submonoid.lean,Mathlib/Deprecated/Subring.lean,Mathlib/FieldTheory/IntermediateField/Basic.lean,Mathlib/GroupTheory/ArchimedeanDensely.lean,Mathlib/GroupTheory/DoubleCoset.lean,Mathlib/GroupTheory/Finiteness.lean,Mathlib/GroupTheory/GroupAction/SubMulAction.lean,Mathlib/LinearAlgebra/AffineSpace/AffineSubspace.lean,Mathlib/LinearAlgebra/Span.lean,Mathlib/RingTheory/Ideal/Operations.lean,Mathlib/RingTheory/NonUnitalSubring/Basic.lean,Mathlib/RingTheory/NonUnitalSubsemiring/Basic.lean,Mathlib/SetTheory/Cardinal/Subfield.lean,Mathlib/Topology/Algebra/Algebra.lean,Mathlib/Topology/Algebra/OpenSubgroup.lean 42 1 ['github-actions'] nobody
254-4303
8 months ago
254-4303
8 months ago
0-0
0 seconds
12617 mans0954
author:mans0954
feat(Algebra/Ring/Defs): Add NonUnitalCommSemiring.toNonUnitalNonAssocCommSemiring instance Adds missing `CommSemiring.toNonUnitalNonAssocCommSemiring` instance. Required for #7569 (specifically [QuadraticMap.linMulLinSelfPosDef](https://github.com/leanprover-community/mathlib4/pull/7569/files#diff-4b8a995fd51c4cb0a5d0ff6413fa1565f87f697d1b552327cfed2c98a4f62f49R1145) ). Zulip discussion: https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/Adding.20an.20instance.20breaks.20.60Mathlib.2ETactic.2ERing.2EBasic.60 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict
label:t-algebra$
11/1 Mathlib/Algebra/Ring/Defs.lean,Mathlib/Tactic/Ring/Basic.lean 2 5 ['eric-wieser', 'github-actions', 'mans0954'] nobody
253-56034
8 months ago
253-56034
8 months ago
147-10606
147 days
7516 ADedecker
author:ADedecker
perf: use `abbrev` to prevent unifying useless data --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP 4/3 Mathlib/Topology/ContinuousFunction/Bounded.lean 1 3 ['ADedecker', 'leanprover-bot', 'mattrobball'] nobody
252-62363
8 months ago
252-62363
8 months ago
0-0
0 seconds
16215 adomasbaliuka
author:adomasbaliuka
feat(Tactic/Linter): lint unwanted unicode Add a text-based style linter that checks all unicode characters. - Only allow whitelisted characters, with a suggestion to add the flagged character to the whitelist - Some characters are specified to use emoji-variant or text-variant. The linter ensures these variant-selectors only appear in the correct places and provides an auto-fix to clean them up. --- Discussed at [Zulip](https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/Whitelist.20for.20Unicode.3F/near/448721083) The current proposal checks each character against a whitelist. There is also the question of what the whitelist should contain. A reasonable whitelist might be "all unicode currently in Mathlib" ∪ [Wikipedia/Mathematical_operators_and_symbols_in_Unicode](https://en.wikipedia.org/wiki/Mathematical_operators_and_symbols_in_Unicode) ∪ [EdAyers/mathlib3/docs/unicode.md](https://github.com/EdAyers/mathlib/blob/fb5c2ffe917049959597b0a93b872e91f4004922/docs/unicode.md). Currently implemented is a subset of this list closer to what's currently present in mathlib. - [x] depends on: #17068 - [x] depends on: #17116 - [ ] depends on: #17129 (part 1 of this PR) - [ ] depends on: #17131 (part 2 of this PR) - Future note: @adomasbaliuka says: "we might add something to the Mathlib 4 docs about this as well?" [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-linter merge-conflict blocked-by-other-PR 462/15 Mathlib/GroupTheory/GroupExtension/Defs.lean,Mathlib/Tactic/Linter/TextBased.lean,Mathlib/Tactic/Linter/UnicodeLinter.lean,Mathlib/Tactic/Widget/Calc.lean,Mathlib/Tactic/Widget/CongrM.lean,Mathlib/Tactic/Widget/Conv.lean,Mathlib/Tactic/Widget/GCongr.lean,Mathlib/Topology/ContinuousFunction/Weierstrass.lean,test/LintStyle.lean 9 51 ['adomasbaliuka', 'eric-wieser', 'github-actions', 'grunweg', 'joneugster', 'mathlib4-dependent-issues-bot'] nobody
252-60370
8 months ago
252-60370
8 months ago
12-19694
12 days
17127 FR-vdash-bot
author:FR-vdash-bot
chore: remove global `Quotient.mk` `⟦·⟧` notation --- Merge this PR when we are ready to migrate to `QuotLike` API (#16421). [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data merge-conflict 137/2 Counterexamples/Pseudoelement.lean,Mathlib/Algebra/Associated/Basic.lean,Mathlib/Algebra/BigOperators/Group/Finset.lean,Mathlib/Algebra/Group/Conj.lean,Mathlib/Algebra/GroupWithZero/NonZeroDivisors.lean,Mathlib/Algebra/Order/CauSeq/Completion.lean,Mathlib/Algebra/Quandle.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Jacobian.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Projective.lean,Mathlib/AlgebraicTopology/FundamentalGroupoid/Basic.lean,Mathlib/AlgebraicTopology/FundamentalGroupoid/FundamentalGroup.lean,Mathlib/AlgebraicTopology/FundamentalGroupoid/InducedMaps.lean,Mathlib/AlgebraicTopology/FundamentalGroupoid/Product.lean,Mathlib/AlgebraicTopology/FundamentalGroupoid/SimplyConnected.lean,Mathlib/CategoryTheory/Abelian/Pseudoelements.lean,Mathlib/CategoryTheory/Limits/Shapes/SingleObj.lean,Mathlib/CategoryTheory/Monoidal/Free/Basic.lean,Mathlib/CategoryTheory/Monoidal/Free/Coherence.lean,Mathlib/CategoryTheory/Skeletal.lean,Mathlib/Data/Finset/Card.lean,Mathlib/Data/Fintype/List.lean,Mathlib/Data/Fintype/Quotient.lean,Mathlib/Data/Multiset/Basic.lean,Mathlib/Data/QPF/Multivariate/Constructions/Fix.lean,Mathlib/Data/QPF/Univariate/Basic.lean,Mathlib/Data/Quot.lean,Mathlib/Data/Real/Basic.lean,Mathlib/Data/Set/Finite.lean,Mathlib/Data/Set/Image.lean,Mathlib/Data/Setoid/Basic.lean,Mathlib/GroupTheory/GroupAction/Basic.lean,Mathlib/GroupTheory/GroupAction/Quotient.lean,Mathlib/LinearAlgebra/Dual.lean,Mathlib/LinearAlgebra/Ray.lean,Mathlib/Logic/Encodable/Basic.lean,Mathlib/Logic/Equiv/Basic.lean,Mathlib/ModelTheory/DirectLimit.lean,Mathlib/ModelTheory/Fraisse.lean,Mathlib/ModelTheory/Quotients.lean,Mathlib/NumberTheory/NumberField/CanonicalEmbedding/FundamentalCone.lean,Mathlib/NumberTheory/NumberField/Embeddings.lean,Mathlib/NumberTheory/NumberField/Units/DirichletTheorem.lean,Mathlib/NumberTheory/Padics/PadicIntegers.lean,Mathlib/NumberTheory/Padics/PadicNumbers.lean,Mathlib/Order/RelIso/Basic.lean,Mathlib/RepresentationTheory/Action/Concrete.lean,Mathlib/SetTheory/Cardinal/Basic.lean,Mathlib/SetTheory/Cardinal/Ordinal.lean,Mathlib/SetTheory/Game/Basic.lean,Mathlib/SetTheory/Game/Birthday.lean,Mathlib/SetTheory/Game/Impartial.lean,Mathlib/SetTheory/Game/Ordinal.lean,Mathlib/SetTheory/Game/State.lean,Mathlib/SetTheory/Lists.lean,Mathlib/SetTheory/Ordinal/Arithmetic.lean,Mathlib/SetTheory/Ordinal/Basic.lean,Mathlib/SetTheory/Surreal/Basic.lean,Mathlib/SetTheory/Surreal/Dyadic.lean,Mathlib/SetTheory/Surreal/Multiplication.lean,Mathlib/SetTheory/ZFC/Basic.lean,Mathlib/SetTheory/ZFC/Rank.lean,Mathlib/Topology/Connected/PathConnected.lean,Mathlib/Topology/Homotopy/HomotopyGroup.lean,Mathlib/Topology/Homotopy/Path.lean,Mathlib/Topology/Homotopy/Product.lean,Mathlib/Topology/MetricSpace/GromovHausdorff.lean,Mathlib/Topology/UniformSpace/Separation.lean,test/interactiveUnfold.lean 68 1 ['github-actions'] nobody
252-57406
8 months ago
252-57406
8 months ago
4-72805
4 days
16888 metinersin
author:metinersin
feat(ModelTheory/Complexity): Define conjunctive and disjunctive normal forms Define `FirstOrder.Language.BoundedFormula.IsDNF` and `FirstOrder.Language.BoundedFormula.IsCNF`. --- - [ ] depends on: #16887 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-logic merge-conflict blocked-by-other-PR 415/7 Mathlib/ModelTheory/Complexity.lean,Mathlib/ModelTheory/Equivalence.lean,Mathlib/ModelTheory/Syntax.lean 3 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
250-1939
8 months ago
250-1939
8 months ago
0-1045
17 minutes
16887 metinersin
author:metinersin
feat(ModelTheory/Complexity): define conjunctive and disjunctive formulas Defines `FirstOrder.Language.BoundedFormula.IsConjunctive` and `FirstOrder.Language.BoundedFormula.IsDisjunctive`. --- - [ ] depends on: #16885 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-logic merge-conflict blocked-by-other-PR 300/7 Mathlib/ModelTheory/Complexity.lean,Mathlib/ModelTheory/Equivalence.lean,Mathlib/ModelTheory/Syntax.lean 3 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
250-1939
8 months ago
250-1940
8 months ago
0-1299
21 minutes
16889 metinersin
author:metinersin
feat(ModelTheory/Complexity): Normal forms Defines `FirstOrder.Language.BoundedFormula.toDNF` and `FirstOrder.Language.BoundedFormula.toCNF` - given a quantifier-free formula, these construct a semantically equivalent formula in disjunctive normal form and conjunctive normal form, respectively. --- - [ ] depends on: #16888 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-logic merge-conflict blocked-by-other-PR 525/7 Mathlib/ModelTheory/Complexity.lean,Mathlib/ModelTheory/Equivalence.lean,Mathlib/ModelTheory/Syntax.lean 3 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
250-1938
8 months ago
250-1938
8 months ago
0-613
10 minutes
14712 FR-vdash-bot
author:FR-vdash-bot
perf: change instance priority and order about `OfNat` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) slow-typeclass-synthesis t-algebra merge-conflict delegated
label:t-algebra$
49/20 Mathlib/Algebra/Group/Nat.lean,Mathlib/Algebra/Group/ZeroOne.lean,Mathlib/Algebra/Homology/Embedding/Basic.lean,Mathlib/Algebra/Tropical/Basic.lean,Mathlib/Data/BitVec.lean,Mathlib/Data/Nat/Cast/Defs.lean,Mathlib/Data/Rat/Defs.lean,Mathlib/Data/UInt.lean,Mathlib/NumberTheory/ArithmeticFunction.lean 9 24 ['FR-vdash-bot', 'MichaelStollBayreuth', 'eric-wieser', 'github-actions', 'j-loreaux', 'leanprover-bot', 'mathlib-bors'] nobody
246-33959
8 months ago
248-57435
8 months ago
20-15089
20 days
11500 mcdoll
author:mcdoll
refactor(Topology/Algebra/Module/WeakDual): Clean up - Move `Dual` and `dualPairing` lower in the import-hierachy - deduplicate `dualPairing` - Bundle continuity statements to `CLM`s. - Make `WeakDual` and `WeakSpace` reducible - Remove `refine'` in favor of `refine` --- Cleaning up `Analysis/NormedSpace/WeakDual` will be done in a second PR [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology merge-conflict awaiting-author 227/179 Mathlib.lean,Mathlib/Analysis/Fourier/RiemannLebesgueLemma.lean,Mathlib/Analysis/InnerProductSpace/Adjoint.lean,Mathlib/Analysis/InnerProductSpace/Dual.lean,Mathlib/Analysis/LocallyConvex/Polar.lean,Mathlib/Analysis/NormedSpace/Dual.lean,Mathlib/Analysis/NormedSpace/WeakDual.lean,Mathlib/Analysis/VonNeumannAlgebra/Basic.lean,Mathlib/MeasureTheory/Function/AEEqOfIntegral.lean,Mathlib/MeasureTheory/Measure/FiniteMeasure.lean,Mathlib/Topology/Algebra/Module/CharacterSpace.lean,Mathlib/Topology/Algebra/Module/Dual.lean,Mathlib/Topology/Algebra/Module/WeakDual.lean,docs/overview.yaml,docs/undergrad.yaml 15 14 ['ADedecker', 'grunweg', 'j-loreaux', 'kkytola', 'mathlib-bors', 'mcdoll'] nobody
244-55902
8 months ago
244-55902
8 months ago
46-5572
46 days
5995 FR-vdash-bot
author:FR-vdash-bot
feat: add APIs about `Quotient.choice` Some docs in this PR refer to the definition in #5576. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data RFC merge-conflict awaiting-author 76/6 Mathlib/Data/Quot.lean 1 3 ['FR-vdash-bot', 'YaelDillies', 'gebner'] eric-wieser
assignee:eric-wieser
243-16148
8 months ago
243-16148
8 months ago
285-35716
285 days
10190 jstoobysmith
author:jstoobysmith
feat(AlgebraicTopology): add Augmented Simplex Category - Added the definition of the category FinLinOrd of finite linear ordered sets. - Added the definition of the augmented simplex category `AugmentedSimplexCategory`, and showed it is the Skeleton of FinLinOrd. - Showed that the category of augmented simplicial objects defined as a comma category is equivalent to the category of functors from `AugmentedSimplexCategory^\op` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra t-topology t-category-theory merge-conflict WIP
label:t-algebra$
720/0 Mathlib.lean,Mathlib/AlgebraicTopology/AugmentedSimplexCategory.lean,Mathlib/AlgebraicTopology/SimplicialObject.lean,Mathlib/Order/Category/FinLinOrd.lean 4 5 ['TwoFX', 'YaelDillies', 'joelriou', 'jstoobysmith'] nobody
243-12137
8 months ago
243-12137
8 months ago
7-63215
7 days
8029 alreadydone
author:alreadydone
refactor: Homotopy between Functions not ContinuousMaps This allows talking about homotopies without needing to supply proofs of continuity for the two ends. This for example simplifies the definition of H-spaces. Of course, if a homotopy exists between two functions, those two functions are automatically continuous because they are restrictions of the homotopy (which is continuous) to subspaces. `Homotopy.refl` still needs a continuous map as input, and `Homotopic` is only an equivalence relation when restricted to ContinuousMap. --- TODO: fix docstrings [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology RFC merge-conflict 246/250 Mathlib/AlgebraicTopology/FundamentalGroupoid/InducedMaps.lean,Mathlib/Topology/Homotopy/Basic.lean,Mathlib/Topology/Homotopy/Contractible.lean,Mathlib/Topology/Homotopy/Equiv.lean,Mathlib/Topology/Homotopy/HSpaces.lean,Mathlib/Topology/Homotopy/HomotopyGroup.lean,Mathlib/Topology/Homotopy/Path.lean,Mathlib/Topology/Homotopy/Product.lean 8 3 ['alreadydone', 'urkud'] nobody
242-86211
7 months ago
335-23470
11 months ago
9-20043
9 days
14627 Multramate
author:Multramate
feat(AlgebraicGeometry/EllipticCurve/Affine): add equivalences between points and explicit WithZero types --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebraic-geometry t-number-theory merge-conflict awaiting-author 159/52 Mathlib/AlgebraicGeometry/EllipticCurve/Affine.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Group.lean 2 9 ['Multramate', 'Ruben-VandeVelde', 'github-actions'] nobody
241-22293
7 months ago
241-22293
7 months ago
46-57206
46 days
15916 vihdzp
author:vihdzp
feat(SetTheory/Ordinal/CantorNormalForm): Coefficients of CNF as finsupp We introduce `CNF_coeff b o e`, which returns the coefficient of `b^e` in the Cantor Normal Form of `o`. --- - [ ] depends on: #15915 I'm not sure if `CNF_Alist` and `CNF_coeff` adhere to naming conventions. Naming suggestions welcome. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-logic merge-conflict blocked-by-other-PR 152/60 Mathlib/SetTheory/Ordinal/CantorNormalForm.lean,Mathlib/SetTheory/Ordinal/Exponential.lean 2 2 ['github-actions', 'leanprover-community-mathlib4-bot'] nobody
240-83370
7 months ago
240-83370
7 months ago
0-542
9 minutes
14619 Command-Master
author:Command-Master
chore: Merge `Trunc` to `Squash` Remove `Trunc` and use `Squash` instead --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor merge-conflict WIP 197/211 Mathlib/CategoryTheory/EpiMono.lean,Mathlib/CategoryTheory/Preadditive/Biproducts.lean,Mathlib/Data/DFinsupp/Basic.lean,Mathlib/Data/Fintype/Basic.lean,Mathlib/Data/Fintype/Card.lean,Mathlib/Data/Fintype/Option.lean,Mathlib/Data/Fintype/Perm.lean,Mathlib/Data/Fintype/Quotient.lean,Mathlib/Data/Quot.lean,Mathlib/Data/Semiquot.lean,Mathlib/GroupTheory/Perm/Cycle/Factors.lean,Mathlib/GroupTheory/Perm/Sign.lean,Mathlib/Logic/Equiv/List.lean 13 3 ['Command-Master', 'github-actions', 'vihdzp'] nobody
240-48489
7 months ago
325-20233
10 months ago
0-0
0 seconds
13156 erdOne
author:erdOne
refactor(Algebra/Module/LocalizedModule): Redefine `LocalizedModule` in terms of `OreLocalization`. --- - [x] depends on: #13151 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict
label:t-algebra$
519/628 Mathlib.lean,Mathlib/Algebra/Module/LocalizedModule.lean,Mathlib/AlgebraicGeometry/Modules/Tilde.lean,Mathlib/RingTheory/DedekindDomain/Different.lean,Mathlib/RingTheory/Localization/BaseChange.lean,Mathlib/RingTheory/OreLocalization/Basic.lean,Mathlib/RingTheory/OreLocalization/Module.lean,Mathlib/RingTheory/OreLocalization/Ring.lean 8 4 ['github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'mattrobball'] nobody
238-23288
7 months ago
238-23288
7 months ago
51-84473
51 days
16348 urkud
author:urkud
refactor(Topology): require `LinearOrder` with `OrderTopology` While the definition formally makes sense for a preorder, this topology is usually not the right one for a non-linear order (e.g., `Real × Real`). See [Zulip thread](https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/Open.20Ioi) --- This PR doesn't cleanup any API, I'm going to do it in a later PR. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order t-topology merge-conflict awaiting-author 33/46 Mathlib/Analysis/Asymptotics/SuperpolynomialDecay.lean,Mathlib/Topology/Algebra/Order/LiminfLimsup.lean,Mathlib/Topology/Instances/Sign.lean,Mathlib/Topology/Order/Basic.lean,Mathlib/Topology/Order/Filter.lean,Mathlib/Topology/Order/MonotoneContinuity.lean 6 10 ['YaelDillies', 'github-actions', 'jcommelin', 'urkud'] nobody
238-22912
7 months ago
238-22912
7 months ago
3-83049
3 days
6034 mattrobball
author:mattrobball
feat (Mathlib.Tactic.FieldSimp) : discharger uses normCast Use `normCast` to assist the discharger in `fieldSimp`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta merge-conflict awaiting-author 30/11 Mathlib/Analysis/Analytic/Composition.lean,Mathlib/Analysis/Fourier/AddCircle.lean,Mathlib/NumberTheory/Modular.lean,Mathlib/RingTheory/RootsOfUnity/Complex.lean,Mathlib/Tactic/FieldSimp.lean,test/FieldSimp.lean 6 7 ['github-actions', 'grunweg', 'mattrobball'] nobody
238-19669
7 months ago
238-19669
7 months ago
1-81851
1 day
13965 pechersky
author:pechersky
feat(Data/DigitExpansion): reals via digit expansion are complete --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) - [ ] depends on: #13964 t-data merge-conflict blocked-by-other-PR 3876/0 Mathlib.lean,Mathlib/Data/DigitExpansion/Add.lean,Mathlib/Data/DigitExpansion/Defs.lean,Mathlib/Data/DigitExpansion/Hensel.lean,Mathlib/Data/DigitExpansion/Integer/Basic.lean,Mathlib/Data/DigitExpansion/Integer/Mul.lean,Mathlib/Data/DigitExpansion/Real/Basic.lean,Mathlib/Data/DigitExpansion/Real/CompleteSpace.lean,Mathlib/Data/DigitExpansion/Real/ConditionallyComplete.lean,docs/references.bib 10 4 ['github-actions', 'leanprover-community-mathlib4-bot'] nobody
236-60080
7 months ago
236-60080
7 months ago
0-0
0 seconds
17519 grunweg
author:grunweg
feat: the `metrisableSpace` linter Similar to #10235, lint on occurrences of `MetricSpace` which should be `MetrisableSpace`. --- - [ ] depends on: #10235 (for all the details) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-linter merge-conflict blocked-by-other-PR 155/21 Mathlib.lean,Mathlib/Algebra/MvPolynomial/PDeriv.lean,Mathlib/AlgebraicGeometry/EllipticCurve/NormalForms.lean,Mathlib/Computability/Halting.lean,Mathlib/Computability/TuringMachine.lean,Mathlib/Data/Fintype/Card.lean,Mathlib/Data/MLList/Split.lean,Mathlib/GroupTheory/Perm/DomMulAct.lean,Mathlib/Logic/Basic.lean,Mathlib/Logic/Encodable/Basic.lean,Mathlib/MeasureTheory/Covering/VitaliFamily.lean,Mathlib/MeasureTheory/Measure/Doubling.lean,Mathlib/NumberTheory/JacobiSum/Basic.lean,Mathlib/Order/Heyting/Regular.lean,Mathlib/Tactic.lean,Mathlib/Tactic/FunProp/RefinedDiscrTree.lean,Mathlib/Tactic/Linter/UnusedAssumptionInType.lean,Mathlib/Util/Superscript.lean,scripts/noshake.json 19 4 ['github-actions', 'mathlib4-dependent-issues-bot', 'urkud'] nobody
235-82994
7 months ago
244-83468
8 months ago*
244-83445
244 days*
16984 hrmacbeth
author:hrmacbeth
feat: extend `module` tactic to handle multiple rings, not strictly ordered by inclusion The `module` tactic currently in Mathlib handles scalars from multiple rings, but only if for any two rings `R` and `S` which appear, either `R` is an algebra over `S` or vice versa. This PR extends the tactic by providing a syntax `module T`, which will handle scalars from any ring `R` which `T` is an algebra over. For example, ```lean example : (2:ℤ) • x = (2:ℚ≥0) • x := by module ``` fails since `ℤ` is not a `ℚ≥0`-algebra and `ℚ≥0` is not a `ℤ`-algebra, but ```lean example : (2:ℤ) • x = (2:ℚ≥0) • x := by module ℚ ``` works since `ℚ` is both a `ℤ`-algebra and a `ℚ≥0`-algebra. This PR is a quick proof-of-concept implementation, just to record the desired approach and tactic syntax. It should not be merged as-is. It has with a lot of code duplication and should be rewritten more efficiently (for example, `parse` and `parseEnsuringType` should be merged to a single function, and the `some`/`none` cases in `matchScalarsAux` should be merged to a uniform treatment) before being considered for merging to Mathlib. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta merge-conflict 158/35 Mathlib/Tactic/Module.lean,test/module.lean 2 1 ['github-actions'] nobody
234-45352
7 months ago
234-45352
7 months ago
0-0
0 seconds
12750 Command-Master
author:Command-Master
feat: define Gray code --- Define binary reflected gray code, both as a permutation of `Nat` and as a permutation of `BitVec n`, and prove some theorems about them. Additionally, remove `@[simp]` from `Nat.bit_false` and `Nat.bit_true`, as `bit0` and `bit1` are deprecated, and add some lemmas to `Bits`, `Bitwise` and `Size`. - [ ] depends on: #12751 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data new-contributor merge-conflict awaiting-author blocked-by-other-PR 226/0 Mathlib.lean,Mathlib/Data/Nat/Bits.lean,Mathlib/Data/Nat/Bitwise.lean,Mathlib/Data/Nat/GrayCode.lean,Mathlib/Data/Nat/Size.lean 5 5 ['Rida-Hamadani', 'alreadydone', 'github-actions', 'grunweg', 'leanprover-community-mathlib4-bot'] nobody
232-24596
7 months ago
232-24596
7 months ago
6-8380
6 days
12414 adomani
author:adomani
test: lint and unlint `·` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict 64/14 Archive/Wiedijk100Theorems/CubingACube.lean,Mathlib/Algebra/Module/Submodule/Bilinear.lean,Mathlib/Tactic/Linter/Multigoal.lean,test/Multigoal.lean 4 4 ['adomani', 'github-actions', 'grunweg', 'leanprover-bot'] nobody
230-21137
7 months ago
230-21137
7 months ago
0-0
0 seconds
16925 YnirPaz
author:YnirPaz
feat(SetTheory/Cardinal/Cofinality): aleph index of singular cardinal has infinite cofinality Prove `Ordinal.aleph0_le_cof_of_not_isRegular`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-set-theory merge-conflict WIP 6/0 Mathlib/SetTheory/Cardinal/Cofinality.lean 1 4 ['YnirPaz', 'github-actions', 'vihdzp'] nobody
228-79119
7 months ago
228-79119
7 months ago
2-57220
2 days
17757 vihdzp
author:vihdzp
refactor(*): generalize typeclass assumptions in morphisms We remove all algebraic axioms from the definitions of morphisms (i.e. `→+`, `→*`, etc.) and assume only the necessary data to state them. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict WIP
label:t-algebra$
86/62 Mathlib/Algebra/Group/Hom/Defs.lean,Mathlib/Algebra/GroupWithZero/Hom.lean,Mathlib/Algebra/Order/Ring/Unbundled/Nonneg.lean,Mathlib/Algebra/Ring/Hom/Defs.lean 4 1 ['github-actions'] nobody
227-83865
7 months ago
227-83865
7 months ago
0-0
0 seconds
16647 eric-wieser
author:eric-wieser
feat: partitions of lists The length of this list is the bell numbers. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data t-combinatorics merge-conflict 311/0 Mathlib.lean,Mathlib/Data/List/Partition.lean 2 1 ['github-actions'] nobody
227-41611
7 months ago
227-41611
7 months ago
0-0
0 seconds
17980 robin-carlier
author:robin-carlier
feat(CategoryTheory/Bicategory/Grothendieck): functors between Grothendieck constructions induced by strong natural transforms Generalize the content of `CategoryTheory/Grothendieck` to pseudofunctor and show that a strong oplax natural transformation of pseudofunctors induces a functor between the Grothendieck contsructions, and that the construction preserves composition and identities. --- The proof of `map_comp_eq` is rather slow and needs a slight increase in heartbeats to go through. It’s probably golfable. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory merge-conflict awaiting-author 143/0 Mathlib/CategoryTheory/Bicategory/Grothendieck.lean 1 2 ['github-actions', 'joelriou'] nobody
227-14142
7 months ago
227-14142
7 months ago
0-0
0 seconds
6533 wupr
author:wupr
WIP: feat(GroupTheory/GroupAction/Basic): add pointwise and setwise stabilizers --- _Work in Progress_ [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict WIP
label:t-algebra$
93/0 Mathlib/GroupTheory/GroupAction/Basic.lean 1 0 [] nobody
223-31389
7 months ago
223-31389
7 months ago
0-0
0 seconds
9605 davikrehalt
author:davikrehalt
feat(Data/Finset & List): Add Lemmas for Sorting and Filtering This PR includes several useful lemmas to the Data/Finset and Data/List modules in Lean's mathlib: 1. `toFinset_filter` (List): Shows that filtering commutes with toFinset. 2. `toFinset_is_singleton_implies_replicate` (List): Shows a list with a singleton toFinset is a List.replicate. 3. `filter_sort_commute` (Finset): Sorting and filtering can be interchanged in Finsets. 4. `Sorted.filter` (List): A sorted list stays sorted after filtering. 5. `Sorted.append_largest` (List): Appending the largest element keeps a list sorted. 6. `sort_monotone_map` (Finset): Relates sorting of a Finset after mapping to sorting of a list. 7. `sort_insert_largest` (Finset): Sorting a Finset with an inserted largest element. 8. `sort_range` (Finset): Sorting a range in a Finset equals the corresponding range list. 9. ~~`filter_eval_true` (List): Filtering a list with a predicate always true keeps the list unchanged.~~ 10. ~~`filter_eval_false` (List): Filtering with an always-false predicate gives an empty list.~~ 11. ~~`pairwise_concat` (List): Iff condition for Pairwise relation in concatenated lists (similar to pairwise_join).~~ 12. `list_map_toFinset` (Finset): toFinset commutes with map under injection --- - [x] depends on: #15952 This is my first PR to mathlib, so I'm not too familiar with etiquette's and more specifically there are two proofs in the PR which uses aesop, and I am not sure if it's frowned upon. I kept the aesop in there for now as I couldn't construct very short proofs otherwise. The sort_range function proof was suggested in https://leanprover.zulipchat.com/#narrow/stream/113489-new-members/topic/Computing.20Finset.20sort.20of.20Finset.20range/near/410346731 by Ruben Van de Velde. Thanks for your time for improving this PR. t-data new-contributor merge-conflict please-adopt awaiting-author 71/0 Mathlib/Data/Finset/Basic.lean,Mathlib/Data/Finset/Image.lean,Mathlib/Data/Finset/Sort.lean,Mathlib/Data/List/Sort.lean 4 30 ['YaelDillies', 'davikrehalt', 'eric-wieser', 'github-actions', 'jcommelin', 'leanprover-community-mathlib4-bot', 'urkud', 'vihdzp'] YaelDillies
assignee:YaelDillies
221-82306
7 months ago
248-51097
8 months ago
12-48560
12 days
13514 madvorak
author:madvorak
feat(Computability/ContextFreeGrammar): closure under union - [ ] depends on: #15895 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-computability merge-conflict blocked-by-other-PR 448/4 Mathlib/Computability/ContextFreeGrammar.lean 1 50 ['Rida-Hamadani', 'YaelDillies', 'github-actions', 'leanprover-community-mathlib4-bot', 'madvorak'] nobody
219-35924
7 months ago
219-35924
7 months ago
72-28392
72 days
17518 grunweg
author:grunweg
feat: lint on declarations mentioning `Invertible` or `Unique` Using the same infrastructure as for #10235. Depends on that PR to land first, and also (for the first lint) a zulip discussion if that change is desired/about the best way to enact it. --- - [ ] depends on: #10235 awaiting-zulip t-linter merge-conflict blocked-by-other-PR 149/7 Mathlib.lean,Mathlib/Algebra/MvPolynomial/PDeriv.lean,Mathlib/Computability/Halting.lean,Mathlib/Computability/TuringMachine.lean,Mathlib/Data/Fintype/Card.lean,Mathlib/GroupTheory/Perm/DomMulAct.lean,Mathlib/Logic/Basic.lean,Mathlib/Logic/Encodable/Basic.lean,Mathlib/NumberTheory/JacobiSum/Basic.lean,Mathlib/Order/Heyting/Regular.lean,Mathlib/RingTheory/MvPolynomial/Symmetric/FundamentalTheorem.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter/UnusedAssumptionInType.lean 13 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'mergify'] nobody
219-8657
7 months ago
244-83579
8 months ago*
0-0
0 seconds*
5364 thorimur
author:thorimur
feat: `wlog ... replacing` This allows hypotheses to be removed from the set of generalized hypotheses. E.g. `wlog h : P replacing h'` will remove `h'` from the hypotheses of the type of `this` and from the context of the goal that will suppose `h`. See [zulip](https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/wlog.20.2E.2E.2E.20replacing.20.2E.2E.2E.3F). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta merge-conflict 125/18 Mathlib/Tactic/WLOG.lean,test/wlog.lean 2 2 ['thorimur', 'urkud'] nobody
217-68963
7 months ago
217-68963
7 months ago
0-0
0 seconds
9654 urkud
author:urkud
feat: add `@[mk_eq]` version of `@[mk_iff]` The new attribute generates theorems like ```lean List.chain_eq : @List.Chain = fun {α} R a a_1 => a_1 = [] ∨ ∃ b l, R a b ∧ List.Chain R b l ∧ a_1 = b :: l ``` and is useful to rewrite in a theorem that argues about the properties of an unapplied inductive predicate. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta merge-conflict awaiting-author 63/9 Mathlib/Lean/Meta.lean,Mathlib/Tactic/MkIffOfInductiveProp.lean,test/MkIffOfInductive.lean 3 6 ['Vierkantor', 'github-actions', 'urkud'] nobody
217-68717
7 months ago
217-68717
7 months ago
25-70815
25 days
16704 AntoineChambert-Loir
author:AntoineChambert-Loir
feat(Mathlib.Data.Ordering.Dickson): Dickson orders Dickson orders are a particular class of well founded orders characterized by the fact that every nonempty set has finitely many minimal elements. They appear in the classical theory of Groebner bases because it is easier to prove that some sets are well founded using this property. WiP. In the `tfae` function, property 2 is exactly `Set.PartiallyWellOrderedOn`, so the PR should be rewritten so as to use that property (and not define `IsDickson`). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order merge-conflict WIP 324/0 Mathlib.lean,Mathlib/Data/Ordering/Dickson.lean,scripts/noshake.json 3 9 ['AntoineChambert-Loir', 'b-mehta', 'github-actions'] nobody
217-47274
7 months ago
217-47274
7 months ago
2-84515
2 days
16428 FR-vdash-bot
author:FR-vdash-bot
test use `QuotLike` APIs --- - [ ] depends on: #16421 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data merge-conflict blocked-by-other-PR 1501/564 Mathlib.lean,Mathlib/Algebra/Associated/Basic.lean,Mathlib/Algebra/BigOperators/Associated.lean,Mathlib/Algebra/GCDMonoid/Basic.lean,Mathlib/Algebra/Group/Conj.lean,Mathlib/Algebra/GroupWithZero/NonZeroDivisors.lean,Mathlib/Algebra/Order/CauSeq/Completion.lean,Mathlib/Algebra/Quandle.lean,Mathlib/CategoryTheory/IsomorphismClasses.lean,Mathlib/CategoryTheory/Monoidal/Free/Basic.lean,Mathlib/CategoryTheory/Monoidal/Free/Coherence.lean,Mathlib/CategoryTheory/Skeletal.lean,Mathlib/Data/Finmap.lean,Mathlib/Data/Fintype/Quotient.lean,Mathlib/Data/Multiset/Basic.lean,Mathlib/Data/Multiset/Functor.lean,Mathlib/Data/QPF/Multivariate/Constructions/Fix.lean,Mathlib/Data/QPF/Univariate/Basic.lean,Mathlib/Data/Quot.lean,Mathlib/Data/QuotLike.lean,Mathlib/Data/Real/Basic.lean,Mathlib/Data/Setoid/Basic.lean,Mathlib/GroupTheory/Coset/Basic.lean,Mathlib/GroupTheory/Coset/Defs.lean,Mathlib/GroupTheory/GroupAction/Basic.lean,Mathlib/GroupTheory/GroupAction/ConjAct.lean,Mathlib/GroupTheory/GroupAction/Defs.lean,Mathlib/GroupTheory/QuotientGroup/Basic.lean,Mathlib/GroupTheory/QuotientGroup/Defs.lean,Mathlib/GroupTheory/Subgroup/Center.lean,Mathlib/LinearAlgebra/Quotient/Basic.lean,Mathlib/LinearAlgebra/Quotient/Defs.lean,Mathlib/Logic/Encodable/Basic.lean,Mathlib/Logic/Equiv/Basic.lean,Mathlib/Logic/Relation.lean,Mathlib/Order/RelIso/Basic.lean,Mathlib/SetTheory/Cardinal/Basic.lean,Mathlib/SetTheory/Cardinal/Finite.lean,Mathlib/SetTheory/Game/Basic.lean,Mathlib/SetTheory/Lists.lean,Mathlib/SetTheory/ZFC/Basic.lean,Mathlib/Topology/Inseparable.lean,test/QuotLike.lean 43 2 ['github-actions', 'leanprover-community-mathlib4-bot'] nobody
217-23736
7 months ago
217-23736
7 months ago
0-0
0 seconds
17746 vihdzp
author:vihdzp
feat(SetTheory/Ordinal/Arithmetic): make `IsNormal` a structure This allows us to give names to its fields. We also explain the definition better in the docstring. --- TODO: golf `preAleph_le_of_isLimit` [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-set-theory merge-conflict WIP 32/27 Mathlib/SetTheory/Cardinal/Aleph.lean,Mathlib/SetTheory/Ordinal/Arithmetic.lean,Mathlib/SetTheory/Ordinal/Exponential.lean,Mathlib/SetTheory/Ordinal/FixedPoint.lean 4 1 ['github-actions'] nobody
217-16568
7 months ago
217-16568
7 months ago
14-53585
14 days
16355 Ruben-VandeVelde
author:Ruben-VandeVelde
feat: odd_{add,sub}_one --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-number-theory merge-conflict awaiting-author
label:t-algebra$
12/0 Mathlib/Algebra/Ring/Int.lean,Mathlib/Algebra/Ring/Parity.lean 2 4 ['Ruben-VandeVelde', 'github-actions', 'urkud'] nobody
216-81471
7 months ago
216-81471
7 months ago
0-57608
16 hours
8479 alexjbest
author:alexjbest
feat: use leaff in CI [Leaff](https://github.com/alexjbest/leaff) is an experimental lean-diff tool, this PR is to experiment with adding it as a CI step. --- I'm not sure yet if it is best to have this always run or only run on request (like bench). If it is always run should it post a comment or simply leave its output it the actions log (maybe as a summary object) the current iteration runs and updates a sticky comment with the latest result [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author WIP 340/0 .github/workflows/bors.yml,.github/workflows/build.yml,.github/workflows/build.yml.in,.github/workflows/build_fork.yml 4 11 ['alexjbest', 'github-actions', 'grunweg', 'kim-em', 'mathlib-bors', 'urkud'] nobody
216-72225
7 months ago
216-72239
7 months ago
0-0
0 seconds
8638 alreadydone
author:alreadydone
refactor: noncommutative tensor product Co-authored-by: Eric Wieser Co-authored-by: Jujian Zhang This draft PR currently only generalizes a single file TensorProduct.lean; it allows TensorProduct to be taken over a non-commutative ring. Most of the declarations in TensorProduct.lean are now generalized to the non-commutative setting, and very few are deleted (their commutative version will be restored in another file). Next plans: + Change the namespace in TensorProduct.lean from TensorProduct to NonCommTensorProduct, and remove the #aligns + I plan to use the same notation for the non-commutative and the commutative TensorProduct, and the user will need to `open scoped` different namespaces to use the one of their choice. + Start a new file TensorProduct/Comm.lean, copy the content of TensorProduct.lean on master into it, change the definition TensorProduct to be semi-reducibly defeq to NonCommTensorProduct (in order to support more instances or unify non-defeq instances that become prop-eq in the commutative setting, e.g. we've chosen the R-action on a tensor product over commutative R to come from the left factor, since the action from the right factor is the same), and reuse the NonComm constructions as much as possible. We then change all files that imports TensorProduct.lean to import TensorProduct/Comm.lean instead. Once we do that, mathlib would compile and this PR would be complete. We can gradually generalize other files about tensor products this way. In this PR: `TensorProduct.map` is now defined in terms of `lTensor` and `rTensor` rather than the other way around, which requires moving `lTensor` and `rTensor` up from their original location. The definition of `rid` also becomes more challenging and is moved down. An evident observation is that actions on the domain of AddMonoidHom / LinearMap is really natural in the context of tensor products and Hom-tensor adjunction (`TensorProduct.lift`), not the default actions on the codomain. For example, it allows us to write the "balanced biadditive monoid homs" in #8536 as simply `N →ₗ[R] M →+ P` (where the right R-action on M turns into the left action on `M →+ P`). For this reason, we disable the default instances `AddMonoidHom/LinearMap.module` at the beginning of the file and enable the `AddMonoidHom/LinearMap.domModule` instances instead. (The action on the codomain would be necessary for the non-commutative version of [TensorProduct.lTensorHomToHomLTensor](https://leanprover-community.github.io/mathlib4_docs/Mathlib/LinearAlgebra/TensorProduct.html#TensorProduct.lTensorHomToHomLTensor) (in the form of `P ⊗[R] (M →+ Q) →+ M →+ P ⊗[R] Q`), but I've deleted it for now.) We register actions on the left factor of a tensor product as the default instance, but we also talk about actions on the right factor (`attribute [local instance] rightModule`). The Tensor-Hom adjunction #8495 is now `uncurryEquiv` in this PR. #8519 is now included in this PR and #8584 is now called `lift` in this PR. `CharacterModule.homEquiv` in #8559 can be obtained by combining `liftEquiv` and `flipMop` in this PR (except for a mop). To refactor the commutative tensor product, we'd need to transfer many R^mop-action to R-action and R^mop-LinearMaps to R-LinearMaps, which can be achieved via `Module.compHom` and `LinearMap.restrictScalars` (requires `LinearMap.CompatibleSMul` instance) given `RingEquiv.toOpposite`. `LinearMap.characterfy` and `CharacterModule.cong` could be obtained from `LinearMap.compAddMonoidHom` in this PR. TODO: + Move delarations that belong to other files. + Change docstrings that are no longer accurate. + Fix some argument order to be more natural. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict WIP
label:t-algebra$
793/676 Mathlib/Algebra/Module/LinearMap.lean,Mathlib/GroupTheory/GroupAction/DomAct/Basic.lean,Mathlib/LinearAlgebra/TensorProduct.lean 3 6 ['alreadydone', 'eric-wieser', 'grhkm21', 'jjaassoonn'] nobody
216-21284
7 months ago
335-23470
11 months ago
0-0
0 seconds
14598 Command-Master
author:Command-Master
chore: add typeclasses to unify various `add_top`, `add_eq_top`, etc. Add the four typeclasses `IsTopAbsorbing`, `IsBotAbsorbing`, `NoTopSum`, `NoBotSum`, as additive equivalents for `MulZeroClass` and `NoZeroDivisors`. Add instances of these for `ENNReal`, `WithTop α`, `WithBot α`, `PUnit`, `EReal`, `PartENat`, `Measure`, `Interval` and `Filter`. Also split `Algebra/Order/AddGroupWithTop` to `Algebra/Order/Group/WithTop` and `Algebra/Order/Monoid/WithTop` --- Previous usages of lemmas with quantified names like `WithTop.add_top` have to be changed to just `add_top`. `add_lt_top` is `@[simp]`, in accordance with `ENNReal.add_lt_top` being `@[simp]`. This affects `WithTop.add_lt_top` which previously hadn't been `@[simp]`. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-order t-algebra merge-conflict
label:t-algebra$
264/195 Archive/Wiedijk100Theorems/BallotProblem.lean,Mathlib.lean,Mathlib/Algebra/Order/Group/WithTop.lean,Mathlib/Algebra/Order/GroupWithZero/Canonical.lean,Mathlib/Algebra/Order/Interval/Basic.lean,Mathlib/Algebra/Order/Monoid/Unbundled/Basic.lean,Mathlib/Algebra/Order/Monoid/Unbundled/Defs.lean,Mathlib/Algebra/Order/Monoid/Unbundled/WithTop.lean,Mathlib/Algebra/Order/Monoid/WithTop.lean,Mathlib/Algebra/PUnitInstances/Order.lean,Mathlib/Algebra/Polynomial/Degree/Definitions.lean,Mathlib/Algebra/Polynomial/Monic.lean,Mathlib/Algebra/Tropical/Basic.lean,Mathlib/Analysis/Analytic/Meromorphic.lean,Mathlib/Analysis/Normed/Lp/ProdLp.lean,Mathlib/Analysis/NormedSpace/ENorm.lean,Mathlib/Analysis/SpecialFunctions/JapaneseBracket.lean,Mathlib/Analysis/SpecialFunctions/Log/ENNRealLog.lean,Mathlib/Data/ENNReal/Operations.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/Data/Nat/PartENat.lean,Mathlib/Data/Nat/WithBot.lean,Mathlib/Data/Real/EReal.lean,Mathlib/LinearAlgebra/Lagrange.lean,Mathlib/MeasureTheory/Covering/Differentiation.lean,Mathlib/MeasureTheory/Decomposition/Lebesgue.lean,Mathlib/MeasureTheory/Function/ConditionalExpectation/CondexpL1.lean,Mathlib/MeasureTheory/Function/Jacobian.lean,Mathlib/MeasureTheory/Function/L1Space.lean,Mathlib/MeasureTheory/Function/L2Space.lean,Mathlib/MeasureTheory/Function/LpSeminorm/Basic.lean,Mathlib/MeasureTheory/Function/LpSeminorm/TriangleInequality.lean,Mathlib/MeasureTheory/Function/LpSpace.lean,Mathlib/MeasureTheory/Function/StronglyMeasurable/Basic.lean,Mathlib/MeasureTheory/Function/UniformIntegrable.lean,Mathlib/MeasureTheory/Integral/Bochner.lean,Mathlib/MeasureTheory/Integral/MeanInequalities.lean,Mathlib/MeasureTheory/Integral/SetIntegral.lean,Mathlib/MeasureTheory/Integral/VitaliCaratheodory.lean,Mathlib/MeasureTheory/Measure/Hausdorff.lean,Mathlib/MeasureTheory/Measure/Lebesgue/Basic.lean,Mathlib/MeasureTheory/Measure/LevyProkhorovMetric.lean,Mathlib/MeasureTheory/Measure/MeasureSpace.lean,Mathlib/MeasureTheory/Measure/MeasureSpaceDef.lean,Mathlib/MeasureTheory/Measure/Regular.lean,Mathlib/MeasureTheory/Measure/Typeclasses.lean,Mathlib/NumberTheory/Padics/PadicNumbers.lean,Mathlib/Order/Filter/Pointwise.lean,Mathlib/Probability/Kernel/Defs.lean,Mathlib/Probability/Martingale/Convergence.lean,Mathlib/RingTheory/Multiplicity.lean,Mathlib/RingTheory/MvPowerSeries/NoZeroDivisors.lean,Mathlib/RingTheory/UniqueFactorizationDomain.lean,Mathlib/Topology/EMetricSpace/Defs.lean,Mathlib/Topology/MetricSpace/Bounded.lean,Mathlib/Topology/MetricSpace/HausdorffDistance.lean,Mathlib/Topology/MetricSpace/Lipschitz.lean 57 30 ['Command-Master', 'YaelDillies', 'github-actions'] nobody
215-52872
7 months ago
215-52872
7 months ago
7-45599
7 days
12778 MichaelStollBayreuth
author:MichaelStollBayreuth
perf: decouple algebraic and order hierarchies in type class search Based on the experience gained with [#12680](https://github.com/leanprover-community/mathlib4/pull/12680), this attempts to decouple the algebraic and order hierarchies in type class search. * We lower the priorities of instances like `OrderedSemiring.toSemiring` (which are generated by the `extends` clause with default priority 1000) to 50. * Additionally, we make the default priority available via `open scoped AlgebraOrderInstances` and use that where appropriate. **Motivation:** Looking at instance synthesization traces, it appears that when (e.g.) presented with the goal to find a `Semiring` instance, the algorithm frequently goes down a rabbit hole trying and failing to find order instances. This seems to be caused by the presence of instances like `OrderedSemiring.toSemiring` with default priority, which are tried early in the search, but lead nowhere (after a fairly long time). These instances are created by declarations of the form ```lean class OrderedSemiring (α : Type u) extends Semiring α, OrderedAddCommMonoid α where ... ``` which automatically sets up (among other things) an instance `OrderedSemiring.toSemiring` with default piority. It appears that these instances cannot be removed completely (only locally in a module), so the next best solution is to make them low priority (which is possible also for downstream modules). To provide for situations where these instances are desired, we put a default priority version in the scope `AlgebraOrderInstances`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) slow-typeclass-synthesis t-order t-algebra merge-conflict
label:t-algebra$
306/27 Mathlib/Algebra/Algebra/Subalgebra/Order.lean,Mathlib/Algebra/ContinuedFractions/Computation/ApproximationCorollaries.lean,Mathlib/Algebra/ContinuedFractions/Computation/Approximations.lean,Mathlib/Algebra/Module/Rat.lean,Mathlib/Algebra/Module/Submodule/Order.lean,Mathlib/Algebra/Order/AbsoluteValue.lean,Mathlib/Algebra/Order/Algebra.lean,Mathlib/Algebra/Order/Antidiag/Prod.lean,Mathlib/Algebra/Order/Archimedean/Basic.lean,Mathlib/Algebra/Order/BigOperators/Group/Finset.lean,Mathlib/Algebra/Order/BigOperators/Group/List.lean,Mathlib/Algebra/Order/BigOperators/Group/Multiset.lean,Mathlib/Algebra/Order/BigOperators/Ring/Finset.lean,Mathlib/Algebra/Order/BigOperators/Ring/List.lean,Mathlib/Algebra/Order/BigOperators/Ring/Multiset.lean,Mathlib/Algebra/Order/CauSeq/Basic.lean,Mathlib/Algebra/Order/Chebyshev.lean,Mathlib/Algebra/Order/CompleteField.lean,Mathlib/Algebra/Order/Field/Basic.lean,Mathlib/Algebra/Order/Field/Defs.lean,Mathlib/Algebra/Order/Field/Pi.lean,Mathlib/Algebra/Order/Floor.lean,Mathlib/Algebra/Order/Floor/Div.lean,Mathlib/Algebra/Order/Group/Defs.lean,Mathlib/Algebra/Order/Group/Units.lean,Mathlib/Algebra/Order/GroupWithZero/Canonical.lean,Mathlib/Algebra/Order/Hom/Basic.lean,Mathlib/Algebra/Order/Hom/Monoid.lean,Mathlib/Algebra/Order/Interval/Basic.lean,Mathlib/Algebra/Order/Interval/Set/Instances.lean,Mathlib/Algebra/Order/Invertible.lean,Mathlib/Algebra/Order/Kleene.lean,Mathlib/Algebra/Order/Module/Algebra.lean,Mathlib/Algebra/Order/Module/Defs.lean,Mathlib/Algebra/Order/Module/Pointwise.lean,Mathlib/Algebra/Order/Monoid/Basic.lean,Mathlib/Algebra/Order/Monoid/Canonical/Defs.lean,Mathlib/Algebra/Order/Monoid/Defs.lean,Mathlib/Algebra/Order/Monoid/OrderDual.lean,Mathlib/Algebra/Order/Monoid/Prod.lean,Mathlib/Algebra/Order/Nonneg/Field.lean,Mathlib/Algebra/Order/Nonneg/Ring.lean,Mathlib/Algebra/Order/Pi.lean,Mathlib/Algebra/Order/Positive/Field.lean,Mathlib/Algebra/Order/Positive/Ring.lean,Mathlib/Algebra/Order/Rearrangement.lean,Mathlib/Algebra/Order/Ring/Basic.lean,Mathlib/Algebra/Order/Ring/Defs.lean,Mathlib/Algebra/Order/Ring/InjSurj.lean,Mathlib/Algebra/Order/Ring/Pow.lean,Mathlib/Algebra/Order/Sub/WithTop.lean,Mathlib/Algebra/Order/ToIntervalMod.lean,Mathlib/Algebra/Ring/BooleanRing.lean,Mathlib/AlgebraicGeometry/Morphisms/RingHomProperties.lean,Mathlib/AlgebraicTopology/FundamentalGroupoid/Basic.lean,Mathlib/Analysis/BoundedVariation.lean,Mathlib/Analysis/Complex/UpperHalfPlane/Metric.lean,Mathlib/Analysis/Convex/Basic.lean,Mathlib/Analysis/Convex/Cone/Basic.lean,Mathlib/Analysis/Convex/Cone/Closure.lean,Mathlib/Analysis/Convex/Cone/Pointed.lean,Mathlib/Analysis/Convex/Cone/Proper.lean,Mathlib/Analysis/Convex/Exposed.lean,Mathlib/Analysis/Convex/Extrema.lean,Mathlib/Analysis/Convex/Function.lean,Mathlib/Analysis/Convex/Gauge.lean,Mathlib/Analysis/Convex/GaugeRescale.lean,Mathlib/Analysis/Convex/Hull.lean,Mathlib/Analysis/Convex/Join.lean,Mathlib/Analysis/Convex/Mul.lean,Mathlib/Analysis/Convex/Quasiconvex.lean,Mathlib/Analysis/Convex/SpecificFunctions/Pow.lean,Mathlib/Analysis/Convex/Star.lean,Mathlib/Analysis/Convex/Strict.lean,Mathlib/Analysis/InnerProductSpace/Orientation.lean,Mathlib/Analysis/MeanInequalities.lean,Mathlib/Analysis/SpecialFunctions/Gamma/BohrMollerup.lean,Mathlib/Analysis/SpecialFunctions/Polynomials.lean,Mathlib/Analysis/SpecificLimits/FloorPow.lean,Mathlib/Analysis/SpecificLimits/Normed.lean,Mathlib/Combinatorics/Optimization/ValuedCSP.lean,Mathlib/Combinatorics/Pigeonhole.lean,Mathlib/Combinatorics/SetFamily/FourFunctions.lean,Mathlib/Data/DFinsupp/Lex.lean,Mathlib/Data/DFinsupp/Multiset.lean,Mathlib/Data/DFinsupp/Order.lean,Mathlib/Data/Finset/MulAntidiagonal.lean,Mathlib/Data/Finsupp/Lex.lean,Mathlib/Data/Finsupp/Multiset.lean,Mathlib/Data/Finsupp/Order.lean,Mathlib/Data/Int/Log.lean,Mathlib/Data/Multiset/Antidiagonal.lean,Mathlib/Data/Multiset/Basic.lean,Mathlib/Data/Multiset/Bind.lean,Mathlib/Data/Nat/Cast/Field.lean,Mathlib/Data/Nat/Cast/Order/Basic.lean,Mathlib/Data/Nat/Choose/Bounds.lean,Mathlib/Data/PNat/Factors.lean,Mathlib/Data/Rat/Denumerable.lean,Mathlib/Data/Set/Pointwise/Interval.lean 135 34 ['MichaelStollBayreuth', 'YaelDillies', 'github-actions', 'leanprover-bot'] nobody
215-51775
7 months ago
215-51775
7 months ago
18-19513
18 days
18636 adomani
author:adomani
Test/latest import report dev This PR is a test accompanying #18631. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) CI merge-conflict 147/0 .github/workflows/latest_import.yml,lakefile.lean 2 1 ['github-actions'] nobody
214-40143
7 months ago
214-40143
7 months ago
0-0
0 seconds
16885 metinersin
author:metinersin
feat(ModelTheory/Complexity): define literals Defines `FirstOrder.Language.BoundedFormula.IsLiteral` and `FirstOrder.Language.BoundedFormula.simpleNot` - an auxiliary operation that takes the negation of a formula and does some simplification. --- - [x] depends on: #16800 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-logic merge-conflict awaiting-author 148/5 Mathlib/ModelTheory/Complexity.lean,Mathlib/ModelTheory/Equivalence.lean,Mathlib/ModelTheory/Semantics.lean,Mathlib/ModelTheory/Syntax.lean 4 20 ['YaelDillies', 'awainverse', 'github-actions', 'mathlib4-dependent-issues-bot', 'metinersin'] nobody
213-8993
7 months ago
213-8993
7 months ago
0-19926
5 hours
18716 jjaassoonn
author:jjaassoonn
feat(Algebra/Module/GradedModule): quotient and subgrading - [ ] depends on: #9820 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra awaiting-CI merge-conflict blocked-by-other-PR WIP
label:t-algebra$
997/191 Counterexamples/HomogeneousPrimeNotPrime.lean,Mathlib.lean,Mathlib/Algebra/Group/Subgroup/Defs.lean,Mathlib/Algebra/Module/GradedModule/Basic.lean,Mathlib/Algebra/Module/GradedModule/QuotientGrading.lean,Mathlib/Algebra/Module/GradedModule/Subgrading.lean,Mathlib/AlgebraicGeometry/ProjectiveSpectrum/Topology.lean,Mathlib/RingTheory/GradedAlgebra/Homogeneous/Ideal.lean,Mathlib/RingTheory/GradedAlgebra/Homogeneous/Submodule.lean,Mathlib/RingTheory/GradedAlgebra/Quotient.lean,Mathlib/RingTheory/GradedAlgebra/Radical.lean,scripts/no_lints_prime_decls.txt 12 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
213-8624
7 months ago
213-8624
7 months ago
0-0
0 seconds
18784 erdOne
author:erdOne
feat(AlgebraicGeometry) use `addMorphismPropertyInstances` --- - [ ] depends on: #18785 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebraic-geometry merge-conflict blocked-by-other-PR 435/91 Mathlib.lean,Mathlib/AlgebraicGeometry/Cover/Open.lean,Mathlib/AlgebraicGeometry/Morphisms/Affine.lean,Mathlib/AlgebraicGeometry/Morphisms/ClosedImmersion.lean,Mathlib/AlgebraicGeometry/Morphisms/FinitePresentation.lean,Mathlib/AlgebraicGeometry/Morphisms/FiniteType.lean,Mathlib/AlgebraicGeometry/Morphisms/OpenImmersion.lean,Mathlib/AlgebraicGeometry/Morphisms/Proper.lean,Mathlib/AlgebraicGeometry/Morphisms/QuasiCompact.lean,Mathlib/AlgebraicGeometry/Morphisms/QuasiSeparated.lean,Mathlib/AlgebraicGeometry/Morphisms/RingHomProperties.lean,Mathlib/AlgebraicGeometry/Morphisms/Smooth.lean,Mathlib/AlgebraicGeometry/Morphisms/UniversallyClosed.lean,Mathlib/AlgebraicGeometry/Restrict.lean,Mathlib/CategoryTheory/MorphismProperty/Composition.lean,Mathlib/CategoryTheory/MorphismProperty/Limits.lean,Mathlib/CategoryTheory/MorphismProperty/Tactic.lean,MathlibTest/AddMorphismPropertyInstances.lean 18 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
212-34045
7 months ago
212-34045
7 months ago
0-1869
31 minutes
9341 winstonyin
author:winstonyin
feat: Naturality of integral curves Let `v` and `v'` be sections of the tangent bundle of manifolds `M` and `M'`, respectively, and let `f : M → M'` be a differentiable map. Then `f` maps integral curves of `v` to integral curves of `v'` if and only if `v` and `v'` are `f`-related. - [x] depends on: #8483 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-differential-geometry merge-conflict awaiting-author 45/0 Mathlib/Geometry/Manifold/IntegralCurve.lean,Mathlib/Topology/Algebra/Module/Basic.lean 2 n/a ['github-actions', 'grunweg', 'leanprover-community-mathlib4-bot', 'winstonyin'] nobody
209-60816
6 months ago
unknown
unknown
16014 vihdzp
author:vihdzp
feat(SetTheory/Ordinal/Principal): even more lemmas on additively principal ordinals --- These are useful for my work on Cantor normal forms. - [ ] depends on: #15989 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-set-theory t-logic merge-conflict blocked-by-other-PR 99/60 Mathlib/SetTheory/Ordinal/Exponential.lean,Mathlib/SetTheory/Ordinal/Principal.lean 2 2 ['github-actions', 'leanprover-community-mathlib4-bot'] nobody
209-32087
6 months ago
209-32087
6 months ago
0-664
11 minutes
7447 BoltonBailey
author:BoltonBailey
feat: reverse for fin tuples The TupleRight section of Data.Fin.Tuple.Basic defines several operations on tuples from the right. This PR redefines these in terms of their from the left counterparts using a new `reverse` function for tuples: ``` cons <-> snoc tail <-> init succ <-> castSucc zero <-> last pred <-> ??? ``` Co-authored-by: Timo Carlin-Burns --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data merge-conflict WIP 112/0 Mathlib/Data/Fin/Tuple/Basic.lean,Mathlib/Data/Fin/Tuple/Reverse.lean 2 0 [] nobody
208-83747
6 months ago
208-83748
6 months ago
0-0
0 seconds
13248 hcWang942
author:hcWang942
feat: basic concepts of auction theory ## Description Formalise some core concepts and results in auction theory: this includes definitions for first-price and second-price auctions, as well as several fundamental results and helping lemmas. This is the very first PR of the project formalizing core concepts and results in auction theory. Our group is working on more contributions on the formalization of game theory prefix. Co-authored-by: Ma Jiajun ## Reference Roughgarden, Tim. ***Twenty Lectures on Algorithmic Game Theory***. Cambridge University Press, 2020. [Link](https://www.cambridge.org/core/books/twenty-lectures-on-algorithmic-game-theory/A9D9427C8F43E7DAEF8C702755B6D72B) --- - [x] Will depend on #14163 once that PR is merged. The Fintype lemmas introduced by this PR have been added in that PR and will be removed from here once that PR gets merged ## Current plan for formalization of Game Theory The current plan for the formalizing of Game Theory include: #### 1. Auction Theory. 🎉 _(200+ lines, this PR)_ - Essential definitions of Sealed-bid auction, First-price auction and Second-price auction. - First-price auction has no dominant strategy. - Second-price auction has dominant strategy. (Second-price auction is DSIC) #### 2. Mechanism design & Myerson's Lemma. 🎉 (400+ lines, pending for modification to Mathlib Standard) - Mechanism design An allocation rule is implementable if there exists - Dominant Strategy Incentive Compatible (DSIC) payment rule - An allocation rule is monotone if for every bidder’s gain is nondecreasing w.r.t. her/his bid - Myerson's Lemma Implementable ⇔ Monotone In the above case, the DSIC payment rule is unique. #### 3. von Neumann‘s Minimax Theorem. 🎉 (800+ lines, pending for modification to Mathlib Standard) - Equilibrium in zero sum game - Formalization strategy: via Loomis’s theorem. #### 4. Nash Equilibrium. 🎉 (pending for modification to Mathlib Standard) #### 5. Brouwer fixed-point theorem. (Work in Progress) #### 6. More Mechanism design. (Planning) new-contributor t-logic merge-conflict awaiting-author 204/0 Mathlib.lean,Mathlib/GameTheory/Auction/Basic.lean,docs/references.bib 3 148 ['Shreyas4991', 'YaelDillies', 'eric-wieser', 'faenuccio', 'github-actions', 'grunweg', 'hcWang942', 'tb65536', 'urkud', 'vihdzp'] hcWang942
assignee:hcWang942
208-47825
6 months ago
unknown
unknown
17675 FR-vdash-bot
author:FR-vdash-bot
perf: do not search algebraic hierarchy when searching `FunLike` hierarchy --- Unification is still very slow. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) slow-typeclass-synthesis t-algebra merge-conflict
label:t-algebra$
144/4 Mathlib.lean,Mathlib/Algebra/Algebra/Equiv.lean,Mathlib/Algebra/Algebra/Hom.lean,Mathlib/Algebra/Algebra/NonUnitalHom.lean,Mathlib/Algebra/Algebra/Rat.lean,Mathlib/Algebra/Group/Equiv/Basic.lean,Mathlib/Algebra/GroupWithZero/Hom.lean,Mathlib/Algebra/Module/Equiv/Defs.lean,Mathlib/Algebra/Module/LinearMap/Defs.lean,Mathlib/Algebra/Order/Hom/Basic.lean,Mathlib/Algebra/Ring/CentroidHom.lean,Mathlib/Algebra/Ring/Equiv.lean,Mathlib/Algebra/Ring/Hom/Defs.lean,Mathlib/Algebra/Star/StarAlgHom.lean,Mathlib/Analysis/Normed/Algebra/Spectrum.lean,Mathlib/Analysis/Normed/Operator/LinearIsometry.lean,Mathlib/GroupTheory/GroupAction/Hom.lean,Mathlib/RingTheory/Bialgebra/Equiv.lean,Mathlib/RingTheory/Bialgebra/Hom.lean,Mathlib/RingTheory/Coalgebra/Equiv.lean,Mathlib/Topology/Algebra/Module/Basic.lean,Mathlib/Util/SetSynthOrder.lean,MathlibTest/TCSynth.lean,scripts/noshake.json 24 5 ['FR-vdash-bot', 'github-actions', 'leanprover-bot'] nobody
208-22958
6 months ago
208-22958
6 months ago
0-0
0 seconds
18805 FR-vdash-bot
author:FR-vdash-bot
refactor: deprecate `SemilinearMapClass` --- I'm not sure if we want to do this, but let's see if we can get a speed up from it first. - [ ] depends on: #18755 - [ ] depends on: #18756 - [ ] depends on: #18806 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-bench t-algebra merge-conflict blocked-by-other-PR WIP
label:t-algebra$
546/318 Mathlib/Algebra/Algebra/Hom.lean,Mathlib/Algebra/Algebra/NonUnitalHom.lean,Mathlib/Algebra/Algebra/Rat.lean,Mathlib/Algebra/BigOperators/Balance.lean,Mathlib/Algebra/BigOperators/Expect.lean,Mathlib/Algebra/Category/ModuleCat/Basic.lean,Mathlib/Algebra/Group/Equiv/Basic.lean,Mathlib/Algebra/Group/Units/Equiv.lean,Mathlib/Algebra/GroupWithZero/Hom.lean,Mathlib/Algebra/Module/Equiv/Defs.lean,Mathlib/Algebra/Module/LinearMap/Defs.lean,Mathlib/Algebra/Module/LinearMap/Rat.lean,Mathlib/Algebra/Module/LocalizedModule/Int.lean,Mathlib/Algebra/Module/Submodule/EqLocus.lean,Mathlib/Algebra/Module/Submodule/Equiv.lean,Mathlib/Algebra/Module/Submodule/Ker.lean,Mathlib/Algebra/Module/Submodule/Map.lean,Mathlib/Algebra/Module/Submodule/Range.lean,Mathlib/Algebra/MvPolynomial/Equiv.lean,Mathlib/Algebra/Order/Hom/Monoid.lean,Mathlib/Algebra/Polynomial/AlgebraMap.lean,Mathlib/Algebra/Prime/Lemmas.lean,Mathlib/Algebra/Ring/Divisibility/Basic.lean,Mathlib/Algebra/Ring/Equiv.lean,Mathlib/Analysis/CStarAlgebra/Spectrum.lean,Mathlib/Analysis/LocallyConvex/WeakOperatorTopology.lean,Mathlib/Analysis/Normed/Algebra/Spectrum.lean,Mathlib/Analysis/Normed/Group/Uniform.lean,Mathlib/Analysis/Normed/Operator/LinearIsometry.lean,Mathlib/CategoryTheory/Limits/ConcreteCategory/WithAlgebraicStructures.lean,Mathlib/Combinatorics/Additive/FreimanHom.lean,Mathlib/Data/Complex/BigOperators.lean,Mathlib/FieldTheory/IsAlgClosed/AlgebraicClosure.lean,Mathlib/FieldTheory/SplittingField/Construction.lean,Mathlib/Geometry/Manifold/Instances/Sphere.lean,Mathlib/GroupTheory/GroupAction/Hom.lean,Mathlib/LinearAlgebra/Ray.lean,Mathlib/LinearAlgebra/Span.lean,Mathlib/RingTheory/Bialgebra/Equiv.lean,Mathlib/RingTheory/Flat/Basic.lean,Mathlib/RingTheory/HahnSeries/Addition.lean,Mathlib/RingTheory/Ideal/Norm.lean,Mathlib/RingTheory/Multiplicity.lean,Mathlib/RingTheory/Polynomial/Opposites.lean,Mathlib/RingTheory/RootsOfUnity/Basic.lean,Mathlib/Topology/Algebra/InfiniteSum/Basic.lean,Mathlib/Topology/Algebra/Module/Basic.lean,Mathlib/Topology/Algebra/Module/CharacterSpace.lean,Mathlib/Topology/Algebra/Module/FiniteDimension.lean,Mathlib/Topology/Algebra/Module/StrongTopology.lean,Mathlib/Topology/Algebra/Module/WeakDual.lean,Mathlib/Topology/Algebra/MulAction.lean,Mathlib/Topology/Homeomorph.lean,Mathlib/Topology/MetricSpace/Isometry.lean,scripts/no_lints_prime_decls.txt 55 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
208-22545
6 months ago
208-22545
6 months ago
0-0
0 seconds
9344 erdOne
author:erdOne
feat: Add `AddGroup.FG` -> `Module.Finite ℤ` as instances --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict awaiting-author
label:t-algebra$
4/0 Mathlib/RingTheory/Finiteness.lean 1 4 ['alreadydone', 'erdOne', 'leanprover-bot'] nobody
207-32218
6 months ago
207-32218
6 months ago
0-0
0 seconds
16116 jjdishere
author:jjdishere
feat(Field): add theorems in Stacks Project Chapter 09FA Fields Add theorems in Stacks Project Chapter 09FA Fields that are not in mathlib. Co-authored-by: --- - [x] depends on: #16105 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra merge-conflict WIP
label:t-algebra$
6/2 Mathlib/Algebra/Field/Defs.lean,Mathlib/Algebra/Field/Subfield.lean 2 6 ['github-actions', 'mathlib4-dependent-issues-bot', 'mergify'] nobody
207-9419
6 months ago
208-78227
6 months ago
0-0
0 seconds
12133 ADedecker
author:ADedecker
feat: generalize instIsLowerProd to arbitrary products Also change a bit the proof of the product case to match my own taste, feel free to tell if you prefer the old one. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order t-topology merge-conflict awaiting-author 34/14 Mathlib/Topology/Constructions.lean,Mathlib/Topology/Order/LowerUpperTopology.lean 2 13 ['Ruben-VandeVelde', 'TwoFX', 'github-actions', 'jcommelin', 'mans0954', 'mathlib-bors', 'riccardobrasca'] nobody
206-41972
6 months ago
206-41972
6 months ago
63-69206
63 days
16637 FR-vdash-bot
author:FR-vdash-bot
perf: reorder `extends` of `(Add)Monoid` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict WIP
label:t-algebra$
46/51 Mathlib/Algebra/Algebra/Hom.lean,Mathlib/Algebra/BigOperators/Ring/List.lean,Mathlib/Algebra/GCDMonoid/Basic.lean,Mathlib/Algebra/Group/Defs.lean,Mathlib/Algebra/Group/Ext.lean,Mathlib/Algebra/Group/Opposite.lean,Mathlib/Algebra/Group/Prod.lean,Mathlib/Algebra/Order/Group/Unbundled/Abs.lean,Mathlib/Algebra/Polynomial/Roots.lean,Mathlib/Algebra/Ring/SumsOfSquares.lean,Mathlib/CategoryTheory/Preadditive/FunctorCategory.lean,Mathlib/Data/Finset/NoncommProd.lean,Mathlib/GroupTheory/Congruence/Defs.lean,Mathlib/GroupTheory/Torsion.lean,Mathlib/LinearAlgebra/LinearPMap.lean,Mathlib/LinearAlgebra/TensorProduct/Basic.lean,Mathlib/Order/Filter/Germ/Basic.lean,Mathlib/RingTheory/Bialgebra/Hom.lean,Mathlib/RingTheory/Coalgebra/Hom.lean,Mathlib/RingTheory/TensorProduct/MvPolynomial.lean 20 3 ['FR-vdash-bot', 'github-actions', 'leanprover-bot'] nobody
206-41210
6 months ago
206-41210
6 months ago
1-49655
1 day
17145 Command-Master
author:Command-Master
feat(Archive/Ioi/Ioi2024Q2): a proof of the solution of question 2 from IOI 2024. --- - [x] depends on: #17189 - [x] depends on: #17190 - [ ] depends on: #17191 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import merge-conflict WIP 1013/1 Archive.lean,Archive/Ioi/Ioi2024Q2.lean,Mathlib.lean,Mathlib/Combinatorics/Orbits.lean,Mathlib/Data/List/SplitLengths.lean,Mathlib/Data/List/Transpose.lean,Mathlib/Data/List/Zip.lean,Mathlib/Data/Vector/Basic.lean,Mathlib/Data/Vector/Defs.lean,Mathlib/Data/Vector/MapLemmas.lean,Mathlib/Data/Vector/Transpose.lean,Mathlib/GroupTheory/Perm/Cycle/Basic.lean,Mathlib/Logic/Function/Iterate.lean,Mathlib/Order/Antisymmetrization.lean,Mathlib/Order/Partition/Finpartition.lean 15 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
206-24388
6 months ago
207-71731
6 months ago
0-0
0 seconds
18765 FR-vdash-bot
author:FR-vdash-bot
chore: changing `outParam` of `MulActionSemiHomClass` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict
label:t-algebra$
60/34 Mathlib/Algebra/Algebra/NonUnitalHom.lean,Mathlib/Algebra/Category/ModuleCat/Limits.lean,Mathlib/Algebra/Module/LinearMap/Defs.lean,Mathlib/GroupTheory/GroupAction/Hom.lean 4 4 ['FR-vdash-bot', 'github-actions', 'leanprover-bot'] nobody
205-83871
6 months ago
205-83871
6 months ago
0-0
0 seconds
18793 JovanGerb
author:JovanGerb
Lean pr testing 5948 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict 9/16 Mathlib/Data/Fin/Tuple/Take.lean,Mathlib/Data/List/Indexes.lean,Mathlib/Data/List/OfFn.lean,lake-manifest.json,lakefile.lean,lean-toolchain 6 6 ['JovanGerb', 'github-actions', 'leanprover-bot'] nobody
205-66745
6 months ago
212-8270
7 months ago
0-0
0 seconds
14739 urkud
author:urkud
feat(Measure): add `gcongr` lemmas --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-measure-probability merge-conflict awaiting-author WIP help-wanted 12/8 Mathlib/MeasureTheory/Covering/Differentiation.lean,Mathlib/MeasureTheory/Function/SimpleFunc.lean,Mathlib/MeasureTheory/Integral/SetToL1.lean,Mathlib/MeasureTheory/Measure/MeasureSpace.lean,Mathlib/Probability/Kernel/Disintegration/Density.lean 5 3 ['github-actions', 'kim-em', 'urkud'] nobody
205-40906
6 months ago
205-40906
6 months ago
0-66587
18 hours
15822 kmill
author:kmill
feat: greedy colorings of finite graphs Proves that the greedy coloring only takes `G.maxDegree + 1` colors. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics merge-conflict 159/0 Mathlib/Combinatorics/SimpleGraph/ConcreteColorings.lean 1 1 ['github-actions'] nobody
203-22664
6 months ago
203-22664
6 months ago
0-0
0 seconds
8661 joelriou
author:joelriou
feat(CategoryTheory/Sites): descent of sheaves In this PR, it is shown that the category of sheaves on a site `(C, J)` identifies as a full subcategory of a category of families of sheaves equipped with a descent data (for a family of objects which cover the final object). Under suitable conditions, it shall be shown that this is an equivalence of categories (TODO). --- This shall be split in small PRs later. - [x] depends on: #8622 - [x] depends on: #8632 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory merge-conflict WIP 1396/26 Mathlib.lean,Mathlib/CategoryTheory/Over.lean,Mathlib/CategoryTheory/Sites/CoverPreserving.lean,Mathlib/CategoryTheory/Sites/Descent.lean,Mathlib/CategoryTheory/Sites/EqualizerSheafCondition.lean,Mathlib/CategoryTheory/Sites/InducedTopology.lean,Mathlib/CategoryTheory/Sites/ObjectsCoverTop.lean,Mathlib/CategoryTheory/Sites/Over.lean,Mathlib/CategoryTheory/Sites/SheafHom.lean,Mathlib/CategoryTheory/Sites/Sieves.lean 10 3 ['github-actions', 'leanprover-community-mathlib4-bot'] nobody
203-18192
6 months ago
496-40665
1 year ago
0-0
0 seconds
18806 FR-vdash-bot
author:FR-vdash-bot
refactor: deprecate `MulEquivClass` --- - [x] depends on: #18809 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict
label:t-algebra$
84/72 Mathlib/Algebra/Group/Equiv/Basic.lean,Mathlib/Algebra/Group/Units/Equiv.lean,Mathlib/Algebra/GroupWithZero/Hom.lean,Mathlib/Algebra/GroupWithZero/NonZeroDivisors.lean,Mathlib/Algebra/Module/Equiv/Defs.lean,Mathlib/Algebra/Order/Hom/Monoid.lean,Mathlib/Algebra/Prime/Lemmas.lean,Mathlib/Algebra/Ring/Divisibility/Basic.lean,Mathlib/Algebra/Ring/Equiv.lean,Mathlib/Combinatorics/Additive/FreimanHom.lean,Mathlib/RingTheory/Bialgebra/Equiv.lean,Mathlib/RingTheory/Ideal/Norm.lean,Mathlib/RingTheory/Localization/FractionRing.lean,Mathlib/RingTheory/Multiplicity.lean,Mathlib/Topology/Algebra/InfiniteSum/Basic.lean 15 6 ['FR-vdash-bot', 'github-actions', 'leanprover-bot', 'mathlib4-dependent-issues-bot', 'vihdzp'] nobody
203-9053
6 months ago
203-9053
6 months ago
4-31794
4 days
19055 JLimperg
author:JLimperg
Test precompilation (batteries + aesop) again merge-conflict 9/8 lake-manifest.json,lakefile.lean 2 5 ['JLimperg', 'github-actions', 'leanprover-bot'] nobody
202-86235
6 months ago
202-86235
6 months ago
0-0
0 seconds
10476 shuxuezhuyi
author:shuxuezhuyi
feat(Topology/UniformSpace): define uniform preordered space We define the semi-uniform structure and the uniform preordered space. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology merge-conflict awaiting-author 94/0 Mathlib.lean,Mathlib/Topology/UniformSpace/UniformOrder.lean,docs/references.bib 3 2 ['shuxuezhuyi'] nobody
202-4846
6 months ago
202-4846
6 months ago
10-33091
10 days
17593 FR-vdash-bot
author:FR-vdash-bot
chore(Algebra/Order/GroupWithZero/Unbundled): deprecate useless lemmas, use `ZeroLEOneClass` There are still some useless lemmas that were simply ported from `Algebra.Order.Monoid.Lemmas`, such as just chain an existing lemma with an assumption and lemmas whose assumptions imply `1 ≤ 0`. This PR removes them. Also, some lemmas have both assumptions like `1 < a` `0 < a`. This PR uses `ZeroLEOneClass` to remove redundant assumptions. --- - [ ] depends on: #17623 Ported from https://github.com/leanprover-community/mathlib/pull/16525 and https://github.com/leanprover-community/mathlib/pull/18158 Adapted from #9250. This version is easier to review. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order t-algebra merge-conflict blocked-by-other-PR
label:t-algebra$
188/48 Archive/Wiedijk100Theorems/BuffonsNeedle.lean,Mathlib/Algebra/Order/GroupWithZero/Canonical.lean,Mathlib/Algebra/Order/GroupWithZero/Unbundled.lean,Mathlib/Combinatorics/SimpleGraph/Triangle/Counting.lean,Mathlib/RingTheory/DedekindDomain/FiniteAdeleRing.lean,Mathlib/Topology/Algebra/Order/Field.lean 6 n/a ['FR-vdash-bot', 'github-actions', 'mathlib4-dependent-issues-bot', 'vihdzp'] nobody
201-28188
6 months ago
unknown
unknown
17623 FR-vdash-bot
author:FR-vdash-bot
feat(Algebra/Order/GroupWithZero/Unbundled): add some lemmas Some lemmas in `Algebra.Order.GroupWithZero.Unbundled` have incorrect or unsatisfactory names, or assumptions that can be omitted using `ZeroLEOneClass`. The lemmas added in this PR are versions of existing lemmas that use the correct or better name or `ZeroLEOneClass` to omit an assumption. The original lemmas will be deprecated in #17593. | New name | Old name | |-------------------------|-------------------------| | `mul_le_one_left₀` | `Left.mul_le_one_of_le_of_le` | | `mul_lt_one_of_le_of_lt_left₀` (`0 ≤ ·` version) / `mul_lt_one_of_le_of_lt_of_pos_left` | `Left.mul_lt_of_le_of_lt_one_of_pos` | | `mul_lt_one_of_lt_of_le_left₀` | `Left.mul_lt_of_lt_of_le_one_of_nonneg` | | `mul_le_one_right₀` | `Right.mul_le_one_of_le_of_le` | | `mul_lt_one_of_lt_of_le_right₀` (`0 ≤ ·` version) / `mul_lt_one_of_lt_of_le_of_pos_right` | `Right.mul_lt_one_of_lt_of_le_of_pos` | | `mul_lt_one_of_le_of_lt_right₀` | `Right.mul_lt_one_of_le_of_lt_of_nonneg` | The following lemmas use `ZeroLEOneClass`. | New name | Old name | |-------------------------|-------------------------| | `(Left.)one_le_mul₀` | `Left.one_le_mul_of_le_of_le` | | `Left.one_lt_mul_of_le_of_lt₀` | `Left.one_lt_mul_of_le_of_lt_of_pos` | | `Left.one_lt_mul_of_lt_of_le₀` | `Left.lt_mul_of_lt_of_one_le_of_nonneg` / `one_lt_mul_of_lt_of_le` (still there) | | `(Left.)one_lt_mul₀` | | | `Right.one_le_mul₀` | `Right.one_le_mul_of_le_of_le` | | `Right.one_lt_mul_of_lt_of_le₀` | `Right.one_lt_mul_of_lt_of_le_of_pos` | | `Right.one_lt_mul_of_le_of_lt₀` | `Right.one_lt_mul_of_le_of_lt_of_nonneg` / `one_lt_mul_of_le_of_lt` (still there) / `one_lt_mul` (still there) | | `Right.one_lt_mul₀` | `Right.one_lt_mul_of_lt_of_lt` | --- Split from #17593. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-zulip t-order t-algebra merge-conflict
label:t-algebra$
146/44 Mathlib/Algebra/Order/GroupWithZero/Canonical.lean,Mathlib/Algebra/Order/GroupWithZero/Unbundled.lean 2 11 ['FR-vdash-bot', 'YaelDillies', 'github-actions', 'j-loreaux'] nobody
201-28188
6 months ago
201-28188
6 months ago
33-64877
33 days
18969 alreadydone
author:alreadydone
chore: generalize Module to NonUnitalSemiring --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict WIP
label:t-algebra$
94/75 Mathlib/Algebra/Category/ModuleCat/Presheaf.lean,Mathlib/Algebra/Group/Action/Defs.lean,Mathlib/Algebra/Group/Action/End.lean,Mathlib/Algebra/Group/Action/Prod.lean,Mathlib/Algebra/Group/Action/TypeTags.lean,Mathlib/Algebra/GroupWithZero/Action/Defs.lean,Mathlib/Algebra/Module/Defs.lean,Mathlib/Algebra/Module/Submodule/Defs.lean,Mathlib/Algebra/Polynomial/Div.lean,Mathlib/Algebra/Polynomial/Laurent.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Group.lean,Mathlib/AlgebraicGeometry/Limits.lean,Mathlib/AlgebraicGeometry/ProjectiveSpectrum/Scheme.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Order.lean,Mathlib/Analysis/Distribution/SchwartzSpace.lean,Mathlib/Geometry/Manifold/Instances/Sphere.lean,Mathlib/GroupTheory/CoprodI.lean,Mathlib/LinearAlgebra/FreeModule/IdealQuotient.lean,Mathlib/LinearAlgebra/LinearDisjoint.lean,Mathlib/LinearAlgebra/Matrix/SesquilinearForm.lean,Mathlib/LinearAlgebra/TensorProduct/Submodule.lean,Mathlib/RingTheory/Filtration.lean,Mathlib/RingTheory/Flat/FaithfullyFlat.lean,Mathlib/RingTheory/Ideal/Cotangent.lean,Mathlib/RingTheory/Ideal/Defs.lean,Mathlib/RingTheory/Ideal/Lattice.lean,Mathlib/RingTheory/Ideal/Operations.lean,Mathlib/RingTheory/Ideal/Prod.lean,Mathlib/RingTheory/Presentation.lean,Mathlib/RingTheory/Smooth/Kaehler.lean,Mathlib/RingTheory/TensorProduct/MvPolynomial.lean 31 11 ['alreadydone', 'eric-wieser', 'github-actions', 'leanprover-bot'] nobody
199-51840
6 months ago
199-51840
6 months ago
0-0
0 seconds
19322 adomani
author:adomani
test: rebuild modifying lint A test to see that #19275 really make CI rebuild every file when the `no_lints` file is modified. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict 9/1 lakefile.lean,scripts/no_lints_prime_decls.txt 2 3 ['adomani', 'github-actions', 'leanprover-bot'] nobody
198-74342
6 months ago
198-74342
6 months ago
0-0
0 seconds
16361 vihdzp
author:vihdzp
chore(SetTheory/Ordinal/FixedPointApproximants): golf + better variable management We avoid making `f : α →o α` and `x : α` explicit arguments when not needed. We then golf most theorems in the file. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-set-theory t-logic merge-conflict awaiting-author 68/101 Mathlib/SetTheory/Ordinal/FixedPointApproximants.lean 1 8 ['PhoenixIra', 'YaelDillies', 'github-actions'] nobody
198-47582
6 months ago
198-47582
6 months ago
50-29942
50 days
17624 FR-vdash-bot
author:FR-vdash-bot
feat(Algebra/Order/GroupWithZero/Unbundled): generalize lemmas --- - [ ] depends on: #17623 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order t-algebra merge-conflict blocked-by-other-PR
label:t-algebra$
121/26 Mathlib/Algebra/Order/GroupWithZero/Unbundled.lean 1 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
197-65360
6 months ago
197-65360
6 months ago
0-465
7 minutes
16743 agjftucker
author:agjftucker
feat(Analysis/Calculus/Implicit): define HasStrictDerivAt.implicitFunOfBivariate In [this](https://leanprover.zulipchat.com/#narrow/stream/116395-maths/topic/Implicit.20function.20theorem.20in.20familiar.20form) Zulip thread @Komyyy proved the "familiar" implicit function theorem. Then I wrote a proposal for a Mathlib PR. (Updated) it went: 1. `noncomputable def implicitFunOfBivariate {f : X × Y → Z} {p₀ : X × Y} {fx : X →L[𝕜] Z} {fy : Y ≃L[𝕜] Z} (hf₀ : HasStrictFDerivAt f (fx.coprod fy) p₀) : X → Y := ...` 2. `noncomputable def implicitFunOfBivariate' {f : X → Y → Z} {x₀ : X} {y₀ : Y} {fx : X →L[𝕜] Z} {fy : Y ≃L[𝕜] Z} (hfx : ContDiffAt 𝕜 1 (f · y₀) x₀) (hfy : ContDiffAt 𝕜 1 (f x₀ ·) y₀) (hfx₀ : fderiv 𝕜 (f · y₀) x₀ = fx) (hfy₀ : fderiv 𝕜 (f x₀ ·) y₀ = fy) : X → Y := ...` 3. `theorem image_eq_iff_implicitFunOfBivariate {f : X × Y → Z} {p₀ : X × Y} {fx : X →L[𝕜] Z} {fy : Y ≃L[𝕜] Z} (hf₀ : HasStrictFDerivAt f (fx.coprod fy) p₀) : ∀ᶠ p in 𝓝 p₀, f p = f p₀ ↔ hf₀.implicitFunOfBivariate p.1 = p.2 := ...` 4. `theorem implicitFunOfBivariate_hasStrictFDerivAt {f : X × Y → Z} {x₀ : X} {y₀ : Y} {fx : X →L[𝕜] Z} {fy : Y ≃L[𝕜] Z} (hf₀ : HasStrictFDerivAt f (fx.coprod fy) (x₀, y₀)) : HasStrictFDerivAt hf₀.implicitFunOfBivariate (-fy.symm ∘L fx) x₀ := ...` 5. something on the second derivative (or higher). Although my proposal elicited no response, I am making this micro-PR to address points 1, 3 and 4 since some limited enthusiasm had been shown earlier in that thread (admittedly for another proposal made by another person). I am testing the waters; if this PR gets anywhere I may continue to work on points 2 and 5. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-analysis merge-conflict awaiting-author 132/8 Mathlib/Analysis/Calculus/Implicit.lean,Mathlib/LinearAlgebra/BilinearForm/Orthogonal.lean,Mathlib/LinearAlgebra/Span.lean,Mathlib/Order/Filter/Prod.lean 4 4 ['github-actions', 'sgouezel'] sgouezel
assignee:sgouezel
196-38467
6 months ago
196-38467
6 months ago
63-71154
63 days
18646 jxjwan
author:jxjwan
feat(RingTheory): isotypic components --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra merge-conflict
label:t-algebra$
308/0 Mathlib/Order/CompactlyGenerated/Basic.lean,Mathlib/RingTheory/Isotypic.lean,Mathlib/RingTheory/SimpleModule.lean 3 1 ['github-actions'] nobody
196-30997
6 months ago
196-30997
6 months ago
20-16585
20 days
17513 FR-vdash-bot
author:FR-vdash-bot
perf: do not search algebraic hierarchies when using `map_*` lemmas --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-bench t-algebra merge-conflict WIP
label:t-algebra$
5/3 Mathlib/Algebra/Group/Hom/Defs.lean,Mathlib/GroupTheory/GroupAction/Hom.lean 2 10 ['FR-vdash-bot', 'github-actions', 'grunweg', 'leanprover-bot'] nobody
196-24382
6 months ago
196-24382
6 months ago
4-72589
4 days
17515 FR-vdash-bot
author:FR-vdash-bot
perf: do not need `simp low` now --- - [ ] depends on: #17513 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict blocked-by-other-PR
label:t-algebra$
12/10 Mathlib/Algebra/Group/Hom/Defs.lean,Mathlib/Analysis/SpecialFunctions/Bernstein.lean,Mathlib/GroupTheory/GroupAction/Hom.lean,Mathlib/NumberTheory/LucasLehmer.lean 4 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
196-24381
6 months ago
196-24381
6 months ago
0-380
6 minutes
19212 Julian
author:Julian
feat(LinearAlgebra): add a variable_alias for VectorSpace Taken directly from the variable_alias docs. Zulip: https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/why.20.5Bvariable_alias.5D.20attribute.20is.20not.20used.20in.20Mathlib.3F --- This is the first actual variable alias added to mathlib. I haven't reviewed variable_alias fully, but it seems like there's at least 3 ways they could be distributed in Mathlib: * alongside whatever subfolder they "belong to" (which is what I've tentatively done here) * In a file called `Aliases` somewhere near the thing they alias (which seems less discoverable to me) * In a single file, a la `Mathlib.TrainingWheels` (with some less playful name) which is meant to define a bunch of more "friendly" aliases all in one place. I kind of like the idea of the third thing as a future module but perhaps it can be synthesized if/when there are more aliases? For now as I say I've done the first one, but please let me know if someone prefers something else. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict
label:t-algebra$
25/0 Mathlib.lean,Mathlib/LinearAlgebra/VectorSpace.lean,scripts/noshake.json 3 10 ['Julian', 'PieterCuijpers', 'github-actions', 'urkud'] nobody
195-29627
6 months ago
195-29627
6 months ago
7-68492
7 days
19337 zeramorphic
author:zeramorphic
feat(Data/Finsupp): generalise `Finsupp` to any "zero" value Remove the explicit dependence of `Finsupp` on `[Zero M]`, instead defining `Finsupp'` (better name pending) to be functions that are equal to a fixed value `z : M` cofinitely often. This PR is intended to do the initial work of replacing the definition of `Finsupp` with an instantiation of the more general definition, without adding any appropriate API. If accepted, the API development will follow in later PRs. Issues to consider: - Naming of `Finsupp'.` - Where should `Finsupp'` lemmas go? Do they need their own file/folder under `Data/`? Relevant Zulip threads: - https://leanprover.zulipchat.com/#narrow/channel/217875-Is-there-code-for-X.3F/topic/Finsupp.20generalisations - https://leanprover.zulipchat.com/#narrow/channel/217875-Is-there-code-for-X.3F/topic/Finsupp-like.20partial.20function Comments are welcome. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data merge-conflict 203/83 Archive/Wiedijk100Theorems/Partition.lean,Mathlib/Algebra/MvPolynomial/Basic.lean,Mathlib/Algebra/MvPolynomial/Rename.lean,Mathlib/Algebra/MvPolynomial/Variables.lean,Mathlib/Algebra/Polynomial/Basic.lean,Mathlib/Algebra/Polynomial/Laurent.lean,Mathlib/Data/Finsupp/BigOperators.lean,Mathlib/Data/Finsupp/Defs.lean,Mathlib/Data/Finsupp/Order.lean,Mathlib/Data/Nat/Choose/Multinomial.lean,Mathlib/RingTheory/MvPolynomial/Symmetric/Defs.lean,Mathlib/RingTheory/PowerBasis.lean,scripts/nolints_prime_decls.txt 13 5 ['github-actions', 'vihdzp', 'zeramorphic'] nobody
193-5704
6 months ago
193-5704
6 months ago
4-60621
4 days
16210 FR-vdash-bot
author:FR-vdash-bot
Clean up quotient APIs ~~We may migrate to `Quot` and `IsEquiv` APIs in the future, but it might be a good start to clean up `Quotient` APIs anyway.~~ The diffs in this PR did not include `QuotLike` APIs, but eventually I decided to migrate to `QuotLike` before deprecating some old APIs. This is because some lemmas don't have alternatives that don't use `· ≈ ·`, and the alternatives that use `· ≈ ·` are in the core. See [Zulip](https://leanprover.zulipchat.com/#narrow/stream/113488-general/topic/.60.28.C2.B7.20.E2.89.88.20.C2.B7.29.60.20in.20.60Quotient.60.20APIs/near/466970386). --- - [x] depends on: #16254 - [x] depends on: #16256 - [x] depends on: #16258 - [x] depends on: #16260 - [x] depends on: #16264 - [x] depends on: #16267 - [ ] depends on: #16314 - [x] depends on: #16410 - [x] depends on: #17588 - [x] depends on: #17594 - [x] depends on: #17940 - [ ] depends on: #17941 --- `QuotLike` - [ ] depends on: #16421 - [ ] depends on: #16428 --- [remaining diffs](https://github.com/leanprover-community/mathlib4/compare/FR_quot_now..FR_quot) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data tech debt merge-conflict blocked-by-other-PR 1015/1114 Counterexamples/CliffordAlgebraNotInjective.lean,Mathlib/Algebra/Associated/Basic.lean,Mathlib/Algebra/BigOperators/Group/Finset.lean,Mathlib/Algebra/CharZero/Quotient.lean,Mathlib/Algebra/DirectLimit.lean,Mathlib/Algebra/GCDMonoid/Basic.lean,Mathlib/Algebra/Lie/Free.lean,Mathlib/Algebra/Lie/Quotient.lean,Mathlib/Algebra/Module/Torsion.lean,Mathlib/Algebra/Module/Zlattice/Basic.lean,Mathlib/Algebra/Order/CauSeq/Completion.lean,Mathlib/Algebra/Periodic.lean,Mathlib/Algebra/RingQuot.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Jacobian.lean,Mathlib/AlgebraicGeometry/ProjectiveSpectrum/Scheme.lean,Mathlib/AlgebraicGeometry/ProjectiveSpectrum/StructureSheaf.lean,Mathlib/Analysis/Normed/Group/Quotient.lean,Mathlib/Analysis/Normed/Group/SemiNormedGrp/Kernels.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Angle.lean,Mathlib/CategoryTheory/ConnectedComponents.lean,Mathlib/CategoryTheory/Limits/Shapes/SingleObj.lean,Mathlib/CategoryTheory/Limits/Types.lean,Mathlib/CategoryTheory/Skeletal.lean,Mathlib/CategoryTheory/Subobject/Basic.lean,Mathlib/CategoryTheory/Subobject/FactorThru.lean,Mathlib/CategoryTheory/Subobject/Lattice.lean,Mathlib/Combinatorics/Quiver/ConnectedComponent.lean,Mathlib/Combinatorics/SimpleGraph/Path.lean,Mathlib/Computability/Reduce.lean,Mathlib/Computability/TuringMachine.lean,Mathlib/Data/Countable/Defs.lean,Mathlib/Data/FinEnum.lean,Mathlib/Data/Finite/Basic.lean,Mathlib/Data/Fintype/Basic.lean,Mathlib/Data/Fintype/Card.lean,Mathlib/Data/Fintype/Quotient.lean,Mathlib/Data/List/Cycle.lean,Mathlib/Data/Multiset/Basic.lean,Mathlib/Data/Quot.lean,Mathlib/Data/Set/Image.lean,Mathlib/Data/Setoid/Basic.lean,Mathlib/Data/Setoid/Partition.lean,Mathlib/Data/Sym/Sym2.lean,Mathlib/FieldTheory/IsAlgClosed/AlgebraicClosure.lean,Mathlib/FieldTheory/PerfectClosure.lean,Mathlib/FieldTheory/SplittingField/Construction.lean,Mathlib/GroupTheory/Abelianization.lean,Mathlib/GroupTheory/Commensurable.lean,Mathlib/GroupTheory/CommutingProbability.lean,Mathlib/GroupTheory/Complement.lean,Mathlib/GroupTheory/Congruence/Basic.lean,Mathlib/GroupTheory/Coprod/Basic.lean,Mathlib/GroupTheory/Coset/Basic.lean,Mathlib/GroupTheory/DoubleCoset.lean,Mathlib/GroupTheory/FreeAbelianGroup.lean,Mathlib/GroupTheory/GroupAction/Basic.lean,Mathlib/GroupTheory/GroupAction/ConjAct.lean,Mathlib/GroupTheory/GroupAction/Quotient.lean,Mathlib/GroupTheory/Index.lean,Mathlib/GroupTheory/MonoidLocalization/Basic.lean,Mathlib/GroupTheory/Nilpotent.lean,Mathlib/GroupTheory/PGroup.lean,Mathlib/GroupTheory/Perm/Cycle/Concrete.lean,Mathlib/GroupTheory/QuotientGroup/Basic.lean,Mathlib/GroupTheory/SchurZassenhaus.lean,Mathlib/GroupTheory/Sylow.lean,Mathlib/GroupTheory/Transfer.lean,Mathlib/LinearAlgebra/Alternating/DomCoprod.lean,Mathlib/LinearAlgebra/Dimension/Constructions.lean,Mathlib/LinearAlgebra/InvariantBasisNumber.lean,Mathlib/LinearAlgebra/Isomorphisms.lean,Mathlib/LinearAlgebra/Projectivization/Basic.lean,Mathlib/LinearAlgebra/Quotient.lean,Mathlib/LinearAlgebra/QuotientPi.lean,Mathlib/Logic/Encodable/Basic.lean,Mathlib/MeasureTheory/Constructions/Polish/Basic.lean,Mathlib/MeasureTheory/Function/AEEqFun.lean,Mathlib/MeasureTheory/Group/FundamentalDomain.lean,Mathlib/MeasureTheory/MeasurableSpace/Basic.lean,Mathlib/MeasureTheory/Measure/Haar/Quotient.lean,Mathlib/ModelTheory/DirectLimit.lean,Mathlib/ModelTheory/Fraisse.lean,Mathlib/ModelTheory/Ultraproducts.lean,Mathlib/NumberTheory/NumberField/Embeddings.lean,Mathlib/NumberTheory/NumberField/Units/DirichletTheorem.lean,Mathlib/NumberTheory/Padics/PadicNumbers.lean,Mathlib/NumberTheory/RamificationInertia.lean,Mathlib/Order/Antisymmetrization.lean,Mathlib/Order/Category/PartOrd.lean,Mathlib/Order/Filter/Germ/Basic.lean,Mathlib/Order/Partition/Finpartition.lean,Mathlib/Order/RelIso/Basic.lean,Mathlib/RepresentationTheory/GroupCohomology/Hilbert90.lean,Mathlib/RingTheory/AdicCompletion/Algebra.lean,Mathlib/RingTheory/AdicCompletion/Basic.lean,Mathlib/RingTheory/AdicCompletion/Functoriality.lean,Mathlib/RingTheory/AdjoinRoot.lean,Mathlib/RingTheory/Congruence/Basic.lean,Mathlib/RingTheory/Flat/Basic.lean,Mathlib/RingTheory/GradedAlgebra/HomogeneousLocalization.lean 134 6 ['FR-vdash-bot', 'github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot'] nobody
192-12845
6 months ago
280-1926
9 months ago
0-0
0 seconds
16956 Parcly-Taxel
author:Parcly-Taxel
refactor(Order/Interval/Finset/Nat): supersymmetrise API As implored by @b-mehta. t-order merge-conflict awaiting-author 93/48 Mathlib/Algebra/BigOperators/Intervals.lean,Mathlib/Data/Nat/Defs.lean,Mathlib/MeasureTheory/Decomposition/UnsignedHahn.lean,Mathlib/NumberTheory/Divisors.lean,Mathlib/Order/Interval/Finset/Nat.lean,Mathlib/Topology/EMetricSpace/Basic.lean,Mathlib/Topology/MetricSpace/Pseudo/Basic.lean 7 7 ['YaelDillies', 'b-mehta', 'github-actions', 'vihdzp'] nobody
192-12391
6 months ago
248-56517
8 months ago
0-61758
17 hours
9598 AlexKontorovich
author:AlexKontorovich
feat(Analysis/Complex): HasPrimitives on disc We prove that holomorphic functions on discs have primitives. TODO: Extend to holomorphic functions on simply connected domains, and use this to define general complex logarithms. Co-authored by: Ian Jauslin ian.jauslin@rutgers.edu --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis merge-conflict 563/10 Mathlib.lean,Mathlib/Analysis/Asymptotics/Asymptotics.lean,Mathlib/Analysis/Complex/CauchyIntegral.lean,Mathlib/Analysis/Complex/HasPrimitives.lean,Mathlib/Data/Complex/Basic.lean,Mathlib/Order/Interval/Set/UnorderedInterval.lean 6 48 ['AlexKontorovich', 'github-actions', 'grunweg', 'loefflerd', 'sgouezel', 'urkud', 'vbeffara'] urkud
assignee:urkud
191-79007
6 months ago
191-79007
6 months ago
100-57565
100 days
19526 metakunt
author:metakunt
feat:closure properties of numbers that are introspective to polynomials Prove Part 1 of Claim 1.(i) of Theorem 6.1 in https://www3.nd.edu/~andyp/notes/AKS.pdf. ---- Zulip discussion: https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Aks.20primality.20Theorem.206.2E1.20Claim.20.28i.29.20proven new-contributor t-number-theory merge-conflict awaiting-author 57/0 Mathlib.lean,Mathlib/NumberTheory/AKSPrimality.lean 2 10 ['Ruben-VandeVelde', 'github-actions', 'jcommelin', 'kim-em', 'metakunt'] nobody
190-32330
6 months ago
190-32330
6 months ago
0-16072
4 hours
19414 vihdzp
author:vihdzp
feat: Nesbitt's inequality We prove [Nesbitt's inequality](https://en.wikipedia.org/wiki/Nesbitt%27s_inequality) `3 / 2 ≤ a / (b + c) + b / (c + a) + c / (b + a)` for a linearly ordered semifield, by reduction to the AM-HM inequality. --- - [ ] depends on: #19415 - [ ] depends on: #19420 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-algebra merge-conflict awaiting-author blocked-by-other-PR WIP
label:t-algebra$
192/142 Mathlib/Algebra/BigOperators/Fin.lean,Mathlib/Algebra/BigOperators/Finsupp.lean,Mathlib/Algebra/Order/Antidiag/Pi.lean,Mathlib/Algebra/Order/BigOperators/Ring/Finset.lean,Mathlib/Algebra/Order/Field/Defs.lean,Mathlib/Analysis/MeanInequalities.lean,Mathlib/Combinatorics/Enumerative/Catalan.lean,Mathlib/Data/Fin/Tuple/NatAntidiagonal.lean,Mathlib/Data/Fin/Tuple/Reflection.lean,Mathlib/Data/Fintype/BigOperators.lean 10 8 ['YaelDillies', 'github-actions', 'mathlib4-dependent-issues-bot', 'vihdzp'] nobody
189-61105
6 months ago
189-61105
6 months ago
0-481
8 minutes
19420 vihdzp
author:vihdzp
feat: AM-HM inequality We prove the weighted and unweighted AM-HM inequalities in linearly ordered semifields. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict awaiting-author WIP
label:t-algebra$
36/2 Mathlib/Algebra/Order/BigOperators/Ring/Finset.lean,Mathlib/Analysis/MeanInequalities.lean 2 7 ['YaelDillies', 'github-actions', 'vihdzp'] nobody
189-61104
6 months ago
189-61104
6 months ago
0-46682
12 hours
19415 vihdzp
author:vihdzp
chore: move results on `Σ i : Fin n, f i` earlier --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data awaiting-CI merge-conflict 131/145 Mathlib/Algebra/BigOperators/Fin.lean,Mathlib/Algebra/BigOperators/Finsupp.lean,Mathlib/Algebra/MvPolynomial/Equiv.lean,Mathlib/Algebra/Order/Antidiag/Pi.lean,Mathlib/Algebra/Polynomial/EraseLead.lean,Mathlib/AlgebraicTopology/AlternatingFaceMapComplex.lean,Mathlib/Combinatorics/Enumerative/Catalan.lean,Mathlib/Combinatorics/Optimization/ValuedCSP.lean,Mathlib/Data/Fin/Tuple/NatAntidiagonal.lean,Mathlib/Data/Fin/Tuple/Reflection.lean,Mathlib/Data/Fintype/BigOperators.lean,Mathlib/Data/Nat/Choose/Multinomial.lean,Mathlib/LinearAlgebra/LinearIndependent.lean 13 2 ['YaelDillies', 'github-actions'] nobody
189-40518
6 months ago
189-40518
6 months ago
0-0
0 seconds
10332 adri326
author:adri326
feat(Topology/Sets): define regular open sets and their boolean algebra Introduces a new module, `Mathlib.Topology.Sets.RegularOpens`, which defines the `IsRegularOpen s` predicate (`interior (closure s) = s`) and `TopologicalSpace.RegularOpens`, the type of bundled regular open sets (defined as `Heyting.Regular (Opens X)`). A few properties of regular open sets (bundled and unbundled) and `interior (closure s)` are proven, and a pointwise instance of `MulAction` is provided for regular open sets. --- This PR belongs to my series of PRs around my formalization of Rubin's theorem. There are two possible ways to implement `RegularOpens`: - either construct them by hand and show that they form a boolean algebra (better def-eq but more boilerplate code required) - or use `Heyting.Regular` on the heyting algebra of `Opens` inherited from the `Frame` instance on them I first chose to use the former approach, but using the latter cuts the length of the construction of the boolean algebra of regular open sets by 100 lines of code, and allows us to inherit all of the helper lemmas defined for `Heyting.Regular`. The big downside, though, is that an element of `RegularOpens` isn't defined as a bundled regular open set anymore, but rather as an `Opens` set `s` for which `Opens.interior ↑(Opens.interior ↑sᶜ)ᶜ = s`, so I added an alternative constructor `RegularOpens.of` that instead accepts any set `s` for which `IsRegularOpen s` holds. Another minor downside is that coercion to a set takes two coercions instead of one. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology merge-conflict WIP 434/0 Mathlib.lean,Mathlib/Data/Set/Pointwise/SMul.lean,Mathlib/Topology/Sets/Opens.lean,Mathlib/Topology/Sets/RegularOpens.lean,docs/references.bib 5 1 ['adri326'] YaelDillies
assignee:YaelDillies
189-33051
6 months ago
298-32241
9 months ago
0-0
0 seconds
10654 smorel394
author:smorel394
feat(LinearAlgebra/{ExteriorPower,LinearIndependent,TensorPower}): define the exterior powers of a module and prove some of their basic properties This introduces the exterior powers of a module and proves some of their basic properties, in `LinearAlgebra/ExteriorPower/Basic.lean` and `LinearAlgebra/ExteriorPower/Generators.lean`. It also adds a lemma in `LinearAlgebra/LinearIndependent.lean` (`linearIndependent_of_dualFamily` : if a family of vectors admits a "dual" family of linear forms, then it is linearly independent) and a construction in `LinearAlgebra/TensorPower.lean` (`linearFormOfFamily` : the linear form on the tensor power of `M` obtained by multiplying a family of linear forms on `M`). # Main definitions ## In `LinearAlgebra/ExteriorPower/Basic.lean`: * `ExteriorPower R n M` is the `n`th exterior power of a `R`-module `M`, defined as `LinearMap.range (ExteriorAlgebra.ι R : M →ₗ[R] ExteriorAlgebra R M) ^ n`. We also introduce the notation `Λ[R]^n M` for `ExteriorPower R n M`. * `ExteriorPower.ιMulti` is the canonical alternating map on `M` with values in `Λ[R]^n M`. * `ExteriorPower.map`: functoriality of exterior powers with respect to linear maps between modules. * `ExteriorPower.toTensorPower`: linear map from the `n`th exterior power to the `n`th tensor power (coming from `MultilinearMap.alternatization` via the universal property of exterior powers). ## In `LinearAlgebra/ExteriorPower/Generators.lean`: * `ExteriorPower.BasisOfBasis`: If `b` is a basis of `M` (indexed by a linearly ordered type), the basis of the `n`th exterior power of `M` formed by the `n`-fold exterior products of elements of `b`. # Main theorems ## In `LinearAlgebra/ExteriorPower/Basic.lean`: * The image of `ExteriorPower.ιMulti` spans `Λ[R]^n M`. * `ExteriorPower.liftAlternatingEquiv` (universal property of the `n`th exterior power of `M`): the linear equivalence between linear maps from `Λ[R]^n M` to a module `N` and `n`-fold alternating maps from `M` to `N`. * `ExteriorPower.map_injective_field`: If `f : M →ₗ[R] N` is injective and `R` is a field, then `ExteriorPower.map n f` is injective. * `ExteriorPower.map_surjective`: If `f : M →ₗ[R] N` is surjective, then `ExteriorPower.map n f` is surjective. * `ExteriorPower.mem_exteriorPower_is_mem_finite`: Every element of `Λ[R]^n M` is in the image of `Λ[R]^n P` for some finitely generated submodule `P` of `M`. ## In `LinearAlgebra/ExteriorPower/Generators.lean`: * `ExteriorPower.Finite`: The `n`th exterior power of a finite module is a finite module. * `ExteriorPower.span_top_of_span_top` and `ExteriorPower.span_top_of_span_top'`: If a family of vectors spans `M`, then the family of its `n`-fold exterior products spans `Λ[R]^n M`. (We give versions in the exterior algebra and in the exterior power.) * `ExteriorPower.FreeOfFree`: If `M` is a free module, then so is its `n`th exterior power. * `ExteriorPower.FinrankOfFiniteFree`: If `R` satisfies the strong rank condition and `M` is finite free of rank `r`, then the `n`th exterior power of `M` is of finrank `Nat.choose r n`. * `ExteriorPower.ιMulti_family_linearIndependent_field`: If `R` is a field, and if `v` is a linearly independent family of vectors (indexed by a linearly ordered type), then the family of its `n`-fold exterior products is also linearly independent. - [x] depends on: #10744 - [ ] depends on: #11156 - [x] depends on: #18590 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-algebra merge-conflict please-adopt blocked-by-other-PR
label:t-algebra$
739/0 Mathlib.lean,Mathlib/LinearAlgebra/ExteriorPower/Basic.lean,Mathlib/LinearAlgebra/ExteriorPower/Generators.lean,Mathlib/LinearAlgebra/LinearIndependent.lean,Mathlib/LinearAlgebra/TensorPower.lean 5 45 ['Ruben-VandeVelde', 'YaelDillies', 'bustercopley', 'eric-wieser', 'github-actions', 'joelriou', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'mattrobball', 'smorel394'] eric-wieser
assignee:eric-wieser
186-70624
6 months ago
186-84951
6 months ago
22-67320
22 days
14501 jjaassoonn
author:jjaassoonn
feat: module structure of filtered colimit of abelian groups over filtered colimit of rings This helps defining the module structure of stalks This contribution was inspired by the AIM workshop "Formalizing algebraic geometry" in June 2024. --- - [x] depends on: #15315 [I am going to move the result in the new file] [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) workshop-AIM-AG-2024 t-algebra t-category-theory merge-conflict awaiting-author
label:t-algebra$
439/2 Mathlib/CategoryTheory/Limits/ConcreteCategory/Basic.lean,Mathlib/CategoryTheory/Limits/ConcreteCategory/WithAlgebraicStructures.lean 2 48 ['YaelDillies', 'adamtopaz', 'erdOne', 'github-actions', 'jjaassoonn', 'joelriou', 'kbuzzard', 'leanprover-community-mathlib4-bot'] joelriou
assignee:joelriou
186-36709
6 months ago
186-36709
6 months ago
64-29952
64 days
19097 Vierkantor
author:Vierkantor
chore(Algebra.Polynomial): split `Polynomial/Basic.lean` into smaller files This PR splits `Mathlib.Algebra.Polynomial.Basic` into the following files: * `Polynomial/Defs.lean`: definition and ring structure on `R[X]` * `Polynomial/Module.lean`: module structure on `R[X]` * `Polynomial/Monomial.lean`: merged definition of `monomial`, `X`, `C` into the existing file (this is probably the file you want to import from now on) * `Polynomial/EraseUpdate.lean`: definition of `erase` and `update` * `Polynomial/Sum.lean`: definition of `sum` Initially I added the monomial results to a new file, but ended up merging it with `Monomial.lean` since the two of them merge cleanly. --- - [ ] depends on: #19091 - [x] depends on: #19095 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict blocked-by-other-PR
label:t-algebra$
3109/2500 Mathlib.lean,Mathlib/Algebra/BigOperators/Finsupp.lean,Mathlib/Algebra/MonoidAlgebra/Basic.lean,Mathlib/Algebra/MonoidAlgebra/Defs.lean,Mathlib/Algebra/MonoidAlgebra/Division.lean,Mathlib/Algebra/MonoidAlgebra/Lift.lean,Mathlib/Algebra/MonoidAlgebra/MapDomain.lean,Mathlib/Algebra/MonoidAlgebra/Module.lean,Mathlib/Algebra/MonoidAlgebra/Opposite.lean,Mathlib/Algebra/MonoidAlgebra/Support.lean,Mathlib/Algebra/Polynomial/Basic.lean,Mathlib/Algebra/Polynomial/Cardinal.lean,Mathlib/Algebra/Polynomial/Coeff.lean,Mathlib/Algebra/Polynomial/Defs.lean,Mathlib/Algebra/Polynomial/Degree/Definitions.lean,Mathlib/Algebra/Polynomial/Degree/TrailingDegree.lean,Mathlib/Algebra/Polynomial/EraseUpdate.lean,Mathlib/Algebra/Polynomial/Eval/Defs.lean,Mathlib/Algebra/Polynomial/Eval/Degree.lean,Mathlib/Algebra/Polynomial/Module.lean,Mathlib/Algebra/Polynomial/Monomial.lean,Mathlib/Algebra/Polynomial/Sum.lean,Mathlib/Data/Finsupp/Basic.lean,Mathlib/Data/Finsupp/Defs.lean,Mathlib/Data/Finsupp/Ext.lean,Mathlib/Data/Finsupp/Fintype.lean,Mathlib/Data/Finsupp/Indicator.lean,Mathlib/Data/Finsupp/Notation.lean,Mathlib/Data/Finsupp/Pointwise.lean,Mathlib/Data/Finsupp/SMulWithZero.lean,Mathlib/Data/Finsupp/Single.lean,Mathlib/Data/List/ToFinsupp.lean,Mathlib/LinearAlgebra/Matrix/Charpoly/Eigs.lean,Mathlib/RingTheory/KrullDimension/Basic.lean,Mathlib/RingTheory/Polynomial/Opposites.lean,Mathlib/RingTheory/PowerSeries/Basic.lean,Mathlib/Tactic/ExtractGoal.lean,MathlibTest/Polynomial.lean,MathlibTest/instance_diamonds.lean,scripts/noshake.json 40 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
181-70207
5 months ago
191-3681
6 months ago
0-0
0 seconds
18756 FR-vdash-bot
author:FR-vdash-bot
refactor: deprecate `DistribMulActionSemiHomClass` `MulSemiringActionSemiHomClass` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict
label:t-algebra$
50/28 Mathlib/Algebra/Algebra/NonUnitalHom.lean,Mathlib/Algebra/Module/LinearMap/Defs.lean,Mathlib/GroupTheory/GroupAction/Hom.lean 3 4 ['FR-vdash-bot', 'github-actions', 'leanprover-bot'] nobody
181-57773
5 months ago
181-57773
5 months ago
31-75259
31 days
17071 ScottCarnahan
author:ScottCarnahan
feat : (LinearAlgebra/RootSystem) : Separation, base, cartanMatrix This PR defines an abstract separation structure for roots, together with the associated base and Cartan Matrix. In general, the good properties will follow from additional order hypotheses on the base ring (implemented in a future PR). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict WIP
label:t-algebra$
111/0 Mathlib.lean,Mathlib/LinearAlgebra/RootSystem/Separation.lean 2 1 ['github-actions'] nobody
181-47674
5 months ago
181-47674
5 months ago
20-56416
20 days
19281 Vierkantor
author:Vierkantor
chore(Algebra/{MonoidAlgebra,Polynomial}): algebra structure in `Basic.lean` [As discussed in PR 19205](https://github.com/leanprover-community/mathlib4/pull/19205#discussion_r1848539148) the Algebra structure on `Polynomial` and `MonoidAlgebra` is very fundamental and shouldn't be hidden away. So let's refactor the import hierarchy to make them available in `Basic.lean`. In addition to #19097, this moves the algebra structure on polynomials into `Algebra/Polynomial/Basic.lean` (which will import the other important instances on polynomials), and moves the algebra structure on `MonoidAlgebra`s into `Algebra/MonoidAlgebra/Basic.lean` (moving most of the existing results in that file into `Lemmas.lean`). --- - [ ] depends on: #19097 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict blocked-by-other-PR
label:t-algebra$
3506/2792 Counterexamples/ZeroDivisorsInAddMonoidAlgebras.lean,Mathlib.lean,Mathlib/Algebra/BigOperators/Finsupp.lean,Mathlib/Algebra/FreeAlgebra.lean,Mathlib/Algebra/FreeNonUnitalNonAssocAlgebra.lean,Mathlib/Algebra/MonoidAlgebra/Basic.lean,Mathlib/Algebra/MonoidAlgebra/Defs.lean,Mathlib/Algebra/MonoidAlgebra/Division.lean,Mathlib/Algebra/MonoidAlgebra/Lemmas.lean,Mathlib/Algebra/MonoidAlgebra/Lift.lean,Mathlib/Algebra/MonoidAlgebra/MapDomain.lean,Mathlib/Algebra/MonoidAlgebra/Module.lean,Mathlib/Algebra/MonoidAlgebra/Opposite.lean,Mathlib/Algebra/MonoidAlgebra/Support.lean,Mathlib/Algebra/MvPolynomial/Basic.lean,Mathlib/Algebra/Polynomial/AlgebraMap.lean,Mathlib/Algebra/Polynomial/Basic.lean,Mathlib/Algebra/Polynomial/Cardinal.lean,Mathlib/Algebra/Polynomial/Coeff.lean,Mathlib/Algebra/Polynomial/Defs.lean,Mathlib/Algebra/Polynomial/Degree/Definitions.lean,Mathlib/Algebra/Polynomial/Degree/TrailingDegree.lean,Mathlib/Algebra/Polynomial/EraseUpdate.lean,Mathlib/Algebra/Polynomial/Eval/Defs.lean,Mathlib/Algebra/Polynomial/Eval/Degree.lean,Mathlib/Algebra/Polynomial/Laurent.lean,Mathlib/Algebra/Polynomial/Module.lean,Mathlib/Algebra/Polynomial/Monomial.lean,Mathlib/Algebra/Polynomial/Sum.lean,Mathlib/Algebra/Polynomial/Taylor.lean,Mathlib/Data/Finsupp/Basic.lean,Mathlib/Data/Finsupp/Defs.lean,Mathlib/Data/Finsupp/Ext.lean,Mathlib/Data/Finsupp/Fintype.lean,Mathlib/Data/Finsupp/Indicator.lean,Mathlib/Data/Finsupp/Notation.lean,Mathlib/Data/Finsupp/Pointwise.lean,Mathlib/Data/Finsupp/SMulWithZero.lean,Mathlib/Data/Finsupp/Single.lean,Mathlib/Data/List/ToFinsupp.lean,Mathlib/LinearAlgebra/Matrix/Charpoly/Eigs.lean,Mathlib/RepresentationTheory/Maschke.lean,Mathlib/RingTheory/FiniteType.lean,Mathlib/RingTheory/KrullDimension/Basic.lean,Mathlib/RingTheory/MvPolynomial/Basic.lean,Mathlib/RingTheory/Polynomial/Opposites.lean,Mathlib/RingTheory/Polynomial/Wronskian.lean,Mathlib/RingTheory/PowerSeries/Basic.lean,Mathlib/Tactic/ExtractGoal.lean,MathlibTest/Polynomial.lean,MathlibTest/instance_diamonds.lean,scripts/noshake.json 52 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
181-26550
5 months ago
191-3680
6 months ago
0-0
0 seconds
16391 vihdzp
author:vihdzp
feat(SetTheory/Ordinal/NaturalOps): characterization of natural operations in base `ω` This essentially gives us a characterization of natural addition and multiplication in terms of the base `ω` Cantor normal form. --- - [ ] depends on: #15989 - [ ] depends on: #15991 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-logic merge-conflict blocked-by-other-PR 362/68 Mathlib/SetTheory/Ordinal/Arithmetic.lean,Mathlib/SetTheory/Ordinal/CantorNormalForm.lean,Mathlib/SetTheory/Ordinal/Exponential.lean,Mathlib/SetTheory/Ordinal/NaturalOps.lean,Mathlib/SetTheory/Ordinal/Principal.lean 5 2 ['github-actions', 'leanprover-community-mathlib4-bot'] nobody
179-12759
5 months ago
270-30736
8 months ago
0-106
1 minute
19125 yhtq
author:yhtq
feat: add theorems to transfer `IsGalois` between pairs of fraction rings feat: add theorems to transfer `IsGalois` between pairs of fraction rings. - [x] depends on: #18404 - [x] depends on: #19124 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra merge-conflict
label:t-algebra$
121/0 Mathlib.lean,Mathlib/FieldTheory/Galois/IsFractionRing.lean,Mathlib/RingTheory/Localization/FractionRing.lean 3 3 ['github-actions', 'mathlib4-dependent-issues-bot', 'tb65536'] nobody
178-70242
5 months ago
185-19265
6 months ago
0-4534
1 hour
19046 j-loreaux
author:j-loreaux
feat: define class `SemigroupAction` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict
label:t-algebra$
34/25 Mathlib/Algebra/Category/ModuleCat/Presheaf.lean,Mathlib/Algebra/Category/ModuleCat/Presheaf/Pushforward.lean,Mathlib/Algebra/Group/Action/Defs.lean,Mathlib/Algebra/Group/Action/End.lean,Mathlib/Algebra/Group/Action/Prod.lean,Mathlib/Algebra/Group/Action/TypeTags.lean,Mathlib/Algebra/Polynomial/Laurent.lean,Mathlib/Analysis/Distribution/SchwartzSpace.lean,Mathlib/GroupTheory/CoprodI.lean,Mathlib/LinearAlgebra/FreeModule/IdealQuotient.lean,Mathlib/LinearAlgebra/Matrix/SesquilinearForm.lean 11 7 ['alreadydone', 'github-actions', 'j-loreaux', 'leanprover-bot', 'urkud'] nobody
178-19257
5 months ago
178-19258
5 months ago
6-21105
6 days
18841 hrmacbeth
author:hrmacbeth
chore: change some `linarith`s to `linear_combination`s Change 100 `linarith`s to `linear_combination`s; this is generally a slight speedup. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) - [x] depends on: #18714 (not strictly blocked by this, but the speed comparison will be more informative after it) merge-conflict WIP 106/107 Archive/Imo/Imo1959Q2.lean,Archive/Imo/Imo1988Q6.lean,Archive/Imo/Imo2005Q3.lean,Archive/Imo/Imo2008Q2.lean,Archive/Imo/Imo2008Q3.lean,Archive/Imo/Imo2013Q5.lean,Archive/Imo/Imo2021Q1.lean,Mathlib/Analysis/Analytic/Basic.lean,Mathlib/Analysis/Analytic/Inverse.lean,Mathlib/Analysis/Calculus/BumpFunction/FiniteDimension.lean,Mathlib/Analysis/Complex/AbelLimit.lean,Mathlib/Analysis/Convex/Gauge.lean,Mathlib/Analysis/Convex/Slope.lean,Mathlib/Analysis/Convex/SpecificFunctions/Basic.lean,Mathlib/Analysis/Convex/Uniform.lean,Mathlib/Analysis/Convex/Visible.lean,Mathlib/Analysis/FunctionalSpaces/SobolevInequality.lean,Mathlib/Analysis/Normed/Module/FiniteDimension.lean,Mathlib/Analysis/PSeries.lean,Mathlib/Analysis/SpecialFunctions/Gamma/BohrMollerup.lean,Mathlib/Analysis/SpecialFunctions/Log/Basic.lean,Mathlib/Analysis/SpecialFunctions/Log/Monotone.lean,Mathlib/Analysis/SpecialFunctions/Pow/Deriv.lean,Mathlib/Analysis/SpecialFunctions/Pow/Real.lean,Mathlib/Analysis/SpecificLimits/FloorPow.lean,Mathlib/MeasureTheory/Covering/BesicovitchVectorSpace.lean,Mathlib/MeasureTheory/Measure/Lebesgue/VolumeOfBalls.lean,Mathlib/NumberTheory/Modular.lean,Mathlib/NumberTheory/Transcendental/Liouville/LiouvilleWith.lean,Mathlib/Probability/Distributions/Pareto.lean 30 29 ['github-actions', 'grunweg', 'hrmacbeth', 'jcommelin', 'leanprover-bot', 'mathlib4-dependent-issues-bot'] nobody
177-31168
5 months ago
177-31168
5 months ago
3-30853
3 days
18748 FR-vdash-bot
author:FR-vdash-bot
refactor: deprecate `ContinuousLinearMapClass` --- - [ ] depends on: #18689 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-topology merge-conflict
label:t-algebra$
115/49 Mathlib/Analysis/CStarAlgebra/Spectrum.lean,Mathlib/Analysis/LocallyConvex/WeakOperatorTopology.lean,Mathlib/Analysis/Normed/Algebra/Spectrum.lean,Mathlib/Analysis/Normed/Operator/LinearIsometry.lean,Mathlib/Topology/Algebra/Module/Basic.lean,Mathlib/Topology/Algebra/Module/CharacterSpace.lean,Mathlib/Topology/Algebra/Module/FiniteDimension.lean,Mathlib/Topology/Algebra/Module/StrongTopology.lean,Mathlib/Topology/Algebra/Module/WeakDual.lean,Mathlib/Topology/Homeomorph.lean 10 5 ['FR-vdash-bot', 'github-actions', 'leanprover-bot', 'mathlib4-dependent-issues-bot'] nobody
175-21786
5 months ago
175-21789
5 months ago
0-989
16 minutes
8686 j-loreaux
author:j-loreaux
refactor: allow non-unital `AlgEquiv` This refactors `AlgEquiv` (and `AlgEquivClass`) to incorporate a `map_smul` field instead of `commutes`. This allows us to weaken the type class assumptions on `AlgEquiv` from: ```lean structure AlgEquiv (R A B : Type*) [CommSemiring R] [Semiring A] [Semiring B] [Algebra R A] [Algebra R B] ``` to: ```lean structure AlgEquiv (R A B : Type*) [Add A] [Add B] [Mul A] [Mul B] [SMul R A] [SMul R B] ``` in accordance with the other `Equiv` structures (e.g., `MulEquiv`, `AddEquiv`, `RingEquiv`). This allows us to use `AlgEquiv` for both unital and non-unital (even non-associative) algebra homomorphisms. Note in addition that `StarAlgEquiv` already follows this paradigm. We supply the convenience constructor `AlgEquiv.ofCommutes`, which is marked `inline` and `reducible`, so that users can still provide go via the `commutes` route for constructing and `AlgEquiv` whenever it is more convenient. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict WIP
label:t-algebra$
286/227 Mathlib/Algebra/Algebra/Equiv.lean,Mathlib/Algebra/Algebra/Opposite.lean,Mathlib/Algebra/Algebra/Pi.lean,Mathlib/Algebra/Algebra/Subalgebra/Basic.lean,Mathlib/Algebra/Algebra/Tower.lean,Mathlib/Algebra/Category/AlgebraCat/Basic.lean,Mathlib/Algebra/DualQuaternion.lean,Mathlib/Algebra/MonoidAlgebra/Basic.lean,Mathlib/Algebra/MonoidAlgebra/ToDirectSum.lean,Mathlib/Algebra/Quaternion.lean,Mathlib/Algebra/Star/Free.lean,Mathlib/Algebra/Star/StarAlgHom.lean,Mathlib/Analysis/NormedSpace/LpEquiv.lean,Mathlib/Data/Complex/Module.lean,Mathlib/Data/IsROrC/Basic.lean,Mathlib/Data/Matrix/Basic.lean,Mathlib/Data/Matrix/DualNumber.lean,Mathlib/Data/MvPolynomial/Equiv.lean,Mathlib/Data/MvPolynomial/Rename.lean,Mathlib/Data/Polynomial/AlgebraMap.lean,Mathlib/LinearAlgebra/Matrix/Basis.lean,Mathlib/LinearAlgebra/Matrix/Charpoly/Coeff.lean,Mathlib/LinearAlgebra/Matrix/Reindex.lean,Mathlib/LinearAlgebra/Matrix/ToLin.lean,Mathlib/LinearAlgebra/TensorProduct/Opposite.lean,Mathlib/Logic/Equiv/TransferInstance.lean,Mathlib/RingTheory/FinitePresentation.lean,Mathlib/RingTheory/GradedAlgebra/Basic.lean,Mathlib/RingTheory/Ideal/QuotientOperations.lean,Mathlib/RingTheory/Localization/Basic.lean,Mathlib/RingTheory/MatrixAlgebra.lean,Mathlib/RingTheory/Polynomial/Quotient.lean,Mathlib/RingTheory/PolynomialAlgebra.lean,Mathlib/RingTheory/TensorProduct.lean,Mathlib/Topology/LocallyConstant/Algebra.lean 35 2 ['eric-wieser', 'j-loreaux'] nobody
172-33581
5 months ago
551-82758
1 year ago
0-0
0 seconds
11142 hmonroe
author:hmonroe
feat(ProofTheory): Define logical symbols abstractly; opens new top-level section, drawing from lean4-logic --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-logic merge-conflict awaiting-author 468/1 Mathlib.lean,Mathlib/Data/Fin/VecNotation.lean,Mathlib/ProofTheory/LogicSymbol.lean 3 19 ['PatrickMassot', 'YaelDillies', 'avigad', 'fpvandoorn', 'github-actions'] nobody
171-40988
5 months ago
171-40988
5 months ago
92-18232
92 days
11210 hmonroe
author:hmonroe
Test commit --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP 1950/1 Mathlib.lean,Mathlib/Data/Fin/VecNotation.lean,Mathlib/ProofTheory/Calculus.lean,Mathlib/ProofTheory/FirstOrder/Arith/Language.lean,Mathlib/ProofTheory/FirstOrder/Basic/Syntax/Term.lean,Mathlib/ProofTheory/LogicSymbol.lean,Mathlib/ProofTheory/Matrix.lean,Mathlib/ProofTheory/Semantics.lean,Mathlib/ProofTheory/System.lean,docs/references.bib 10 100 ['github-actions'] nobody
171-40987
5 months ago
171-40987
5 months ago
0-0
0 seconds
19621 Command-Master
author:Command-Master
feat: Multiplicity and prime-adic valuation of derivations --- - [ ] depends on: #19596 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-algebra merge-conflict blocked-by-other-PR
label:t-algebra$
397/13 Mathlib.lean,Mathlib/Algebra/Order/AddGroupWithTop.lean,Mathlib/Algebra/Order/Monoid/Unbundled/WithTop.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/Order/WithBot.lean,Mathlib/RingTheory/Derivation/Multiplicity.lean,Mathlib/RingTheory/DiscreteValuationRing/Basic.lean,Mathlib/RingTheory/Valuation/Basic.lean,Mathlib/RingTheory/Valuation/PrimeMultiplicity.lean 9 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
171-23248
5 months ago
171-23248
5 months ago
0-666
11 minutes
18262 joelriou
author:joelriou
feat(Algebra/Category/ModuleCat/Presheaf): exterior powers of presheaves of modules --- - [x] depends on: #18261 - [ ] depends on: #18236 - [ ] depends on: #18197 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-category-theory merge-conflict blocked-by-other-PR WIP
label:t-algebra$
874/0 Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/ChangeOfRings.lean,Mathlib/Algebra/Category/ModuleCat/ExteriorPower.lean,Mathlib/Algebra/Category/ModuleCat/Presheaf/ExteriorPower.lean,Mathlib/Algebra/Category/ModuleCat/Presheaf/FunctorOfNatTrans.lean,Mathlib/Algebra/Category/ModuleCat/Pseudofunctor.lean 6 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
171-14543
5 months ago
206-81008
6 months ago
0-0
0 seconds
18294 FR-vdash-bot
author:FR-vdash-bot
perf: make `Mul.toSMul` higher priority --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-bench t-algebra merge-conflict
label:t-algebra$
2/5 Mathlib/Algebra/Group/Action/Defs.lean,Mathlib/Algebra/Order/Field/Pointwise.lean,Mathlib/Combinatorics/Additive/AP/Three/Defs.lean,Mathlib/Topology/Algebra/Module/WeakBilin.lean 4 4 ['FR-vdash-bot', 'github-actions', 'leanprover-bot'] nobody
166-22180
5 months ago
166-22181
5 months ago
0-0
0 seconds
19699 vihdzp
author:vihdzp
chore(SetTheory/Cardinal/Basic): tweak `#α = 0`, `#α = 1`, etc. lemmas We rename `le_one_iff_subsingleton` → `mk_le_one_iff` and `mk_le_one_iff_set_subsingleton` → `mk_set_le_one_iff` to match the names of other lemmas in this section. We also add `mk_eq_one_iff` and `mk_set_eq_one_iff`. --- These last two lemmas can probably be golfed somehow. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-set-theory awaiting-CI merge-conflict 48/16 Mathlib/SetTheory/Cardinal/Basic.lean 1 1 ['github-actions'] nobody
164-27614
5 months ago
164-27614
5 months ago
0-5976
1 hour
11156 smorel394
author:smorel394
feat(LinearAlgebra/{TensorProductBasis,Dual}): basis and dual of `PiTensorProduct` Construct a basis of a `PiTensorProduct` of modules given bases of the modules, and relationship between the dual of a `PiTensorProduct` and the `PiTensorProduct` of the duals. Main results: * `Basis.piTensorProduct` (in `LinearAlgebra/TensorProductBasis.lean`): Let `ι` be a `Fintype` and `M` be a family of modules indexed by `ι`. If `b i : κ i → M i` is a basis for every `i` in `ι`, then `fun (p : Π i, κ i) ↦ ⨂ₜ[R] i, b i (p i)` is a basis of `⨂[R] i, M i`. * `PiTensorProduct.dualDistrib` (in `LinearAlgebra/Dual.lean`): The canonical linear map from `⨂[R] i, Dual R (M i)` to `Dual R (⨂[R] i, M i)`, sending `⨂ₜ[R] i, f i` to the composition of `PiTensorProduct.map f` with the linear equivalence `⨂[R] i, R →ₗ R` given by multiplication. * `PiTensorProduct.dualDistribEquiv` (also in `LinearAlgebra/Dual.lean`): A linear equivalence between `⨂[R] i, Dual R (M i)` and `Dual R (⨂[R] i, M i)` when all `M i` are finite free modules. If `f : (i : ι) → Dual R (M i)`, then this equivalence sends `⨂ₜ[R] i, f i` to the composition of `PiTensorProduct.map f` with the natural isomorphism `⨂[R] i, R ≃ R` given by multiplication. - [ ] depends on: #11155 (currently used as the base branch; do not merge without switching it back to `master`!) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import new-contributor t-algebra merge-conflict please-adopt blocked-by-other-PR
label:t-algebra$
166/2 Mathlib/LinearAlgebra/DirectSum/Finsupp.lean,Mathlib/LinearAlgebra/Dual.lean,Mathlib/LinearAlgebra/TensorProduct/Basis.lean 3 4 ['eric-wieser', 'github-actions', 'leanprover-community-mathlib4-bot'] nobody
161-22673
5 months ago
206-38301
6 months ago
0-0
0 seconds
15269 kkytola
author:kkytola
feat: Add ENNReal.floor A right-continuous floor function on `ENNReal`. --- - [x] depends on: #13938 - [ ] depends on: #15773 (general type class for `ENat`-valued floor functions) - [x] depends on: #15380 (topology on `ENat` is needed to state right continuity of the floor function) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order t-algebra merge-conflict awaiting-author blocked-by-other-PR
label:t-algebra$
445/0 Mathlib.lean,Mathlib/Algebra/Order/EFloor.lean,Mathlib/Data/ENNReal/Floor.lean,Mathlib/Data/Nat/Lattice.lean 4 18 ['YaelDillies', 'github-actions', 'kkytola', 'leanprover-community-mathlib4-bot', 'urkud'] nobody
157-81877
5 months ago
157-81877
5 months ago
0-3440
57 minutes
15773 kkytola
author:kkytola
feat: Add type class for ENat-valued floor functions This PR adds a type class for extended natural number -valued floor functions. This is split off from #15269, where the suggestions were to make the floor function on ENNReal ENat-valued and to have an API mimicling FloorSemirings. Besides ENNReal, at least ENNRat would naturally satisfy the general type class. --- Two things are worth noting: * To fully mimic `FloorSemiring` API, also ceiling functions need to be added. The plan is to do that in a later PR. * The PR introduces the class `CastNatENatClass` to ensure that `natCast` and a coercion from `ENat` behave in the natural and order-respecing manner. This feels a little ad hoc, but such assumptions are needed for general `ENat`-valued floor functions to behave well. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order merge-conflict awaiting-author 231/0 Mathlib.lean,Mathlib/Algebra/Order/EFloor.lean,Mathlib/Data/ENat/Basic.lean 3 5 ['YaelDillies', 'github-actions', 'kkytola', 'urkud'] nobody
157-81754
5 months ago
157-81754
5 months ago
66-24436
66 days
3251 kmill
author:kmill
feat: deriving `LinearOrder` for simple enough inductive types Uses the same machinery underlying the `Fintype` derive handler to derive a lexicographical `LinearOrder` for non-recursive inductive types that have no indices. In principle more complicated types can have `LinearOrder`s, but that would require a more sophisticated implementation. --- - [x] depends on: #3198 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta merge-conflict awaiting-author WIP 82/0 Mathlib.lean,Mathlib/Tactic/DeriveLinearOrder.lean 2 5 ['ChrisHughes24', 'kim-em', 'kmill', 'vihdzp'] nobody
155-56407
5 months ago
155-56407
5 months ago
1-80342
1 day
3610 TimothyGu
author:TimothyGu
feat: derive Infinite automatically for inductive types Deals with recursive types, but not mutually recursive types or types with indices right now. See docstring for details. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta merge-conflict awaiting-author 517/0 Mathlib.lean,Mathlib/Tactic/DeriveInfinite.lean,test/DeriveInfinite.lean 3 11 ['TimothyGu', 'digama0', 'eric-wieser', 'grunweg', 'kim-em', 'kmill'] kmill
assignee:kmill
155-56406
5 months ago
155-56406
5 months ago
0-0
0 seconds
16120 awainverse
author:awainverse
feat(ModelTheory/Algebra/Ring/Basic): Ring homomorphisms are a `StrongHomClass` for the language of rings Adds an `IsAlgebraic` instance to the language of rings Adds a `StrongHomClass` instance to the type of ring homomorphisms between rings with `CompatibleRing` structures --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-logic t-algebra RFC merge-conflict
label:t-algebra$
34/13 Mathlib/ModelTheory/Algebra/Ring/Basic.lean 1 10 ['ChrisHughes24', 'YaelDillies', 'awainverse', 'github-actions', 'jcommelin'] nobody
153-73947
5 months ago
153-73947
5 months ago
135-29017
135 days
15045 Command-Master
author:Command-Master
fix(LinearAlgebra/Alternating/Basic): fix `MultilinearMap.alternatization` See https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/kernel.20deep.20recursion.20detected. Fix ```lean import Mathlib.LinearAlgebra.Determinant example : (1 : Matrix (Fin 8) (Fin 8) ℚ).det = 1 := by rw [Matrix.det_one] ``` causing a `(kernel) deep recursion detected` error. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict awaiting-author
label:t-algebra$
51/21 Mathlib/Data/Nat/Factorial/SuperFactorial.lean,Mathlib/LinearAlgebra/Alternating/Basic.lean,test/DetOne.lean 3 12 ['Command-Master', 'PatrickMassot', 'eric-wieser', 'github-actions', 'grhkm21', 'grunweg', 'kbuzzard', 'kim-em'] nobody
153-41236
5 months ago
153-41237
5 months ago
0-8789
2 hours
17471 joelriou
author:joelriou
feat(Algebra/ModuleCat/Differentials/Sheaf): the sheaf of relative differentials --- - [ ] depends on: #17366 - [x] depends on: #17388 - [x] depends on: #16755 - [ ] depends on: #17469 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-algebraic-geometry t-category-theory merge-conflict blocked-by-other-PR WIP 740/10 Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Differentials/Presheaf.lean,Mathlib/Algebra/Category/ModuleCat/Differentials/Sheaf.lean,Mathlib/Algebra/Category/ModuleCat/Presheaf/Limits.lean,Mathlib/Algebra/Category/ModuleCat/Presheaf/Pullback.lean,Mathlib/Algebra/Category/Ring/Constructions.lean,Mathlib/Algebra/Ring/Hom/Defs.lean,Mathlib/AlgebraicGeometry/Modules/Differentials.lean,Mathlib/Geometry/RingedSpace/SheafedSpace.lean 9 n/a ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
149-9894
4 months ago
unknown
unknown
19462 joelriou
author:joelriou
feat(AlgebraicGeometry): étale sheafification After #19096 and #18945 are merged, if `S : Scheme.{u}`, we shall get instances like `HasSheafify (smallEtaleTopology S) (Type (u + 1))` which means that in order to sheafify preshaves over the small étale site of `S`, we need to assume a certain bump in the universe in the target category. With the main result in this PR (there are still a few sorries), we shall get `HasSheafify (smallEtaleTopology S) (Type u)`. Then, in the subsequent development of étale formalism, we can work in `Type u` (or `Ab.{u}`, etc). --- This is a draft. - [ ] depends on: #19444 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebraic-geometry merge-conflict blocked-by-other-PR WIP 1336/2 Mathlib.lean,Mathlib/AlgebraicGeometry/Sites/EtaleSheafification.lean,Mathlib/CategoryTheory/Sites/Continuous.lean,Mathlib/CategoryTheory/Sites/DenseSubsite.lean,Mathlib/CategoryTheory/Sites/LocallyFullyFaithful.lean,Mathlib/CategoryTheory/Sites/OneHypercover.lean,Mathlib/CategoryTheory/Sites/OneHypercoverDense.lean,Mathlib/CategoryTheory/Sites/Sieves.lean 8 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
147-22352
4 months ago
194-30489
6 months ago
0-200
3 minutes
20527 trivial1711
author:trivial1711
refactor(Topology/UniformSpace/Completion): more descriptive names for `α → Completion α` - We rename the various maps `α → Completion α` in order to make their names more consistent. - Let `α` be a uniform space. We rename the uniformly continuous function `α → Completion α` from `UniformSpace.Completion.coe'` to `UniformSpace.Completion.coe`. - Let `α` be a uniform additive group. We rename the additive group homomorphism `α →+ Completion α` from `UniformSpace.Completion.toCompl` to `UniformSpace.Completion.coeAddHom`. - Let `α` be a uniform ring. The ring homomorphism `α →+* Completion α` is called `UniformSpace.Completion.coeRingHom`; its name is unchanged. - Let `α` be a normed space over a field `𝕜`. We rename the linear isometry `α →ₗᵢ[𝕜] Completion α` from `UniformSpace.Completion.toComplₗᵢ` to `UniformSpace.Completion.coeₗᵢ`. - Let `α` be a normed space over a field `𝕜`. We rename the continuous linear map `α →L[𝕜] Completion α` from `UniformSpace.Completion.toComplL` to `UniformSpace.Completion.coeL`. - Let `α` be a normed additive group. We rename the norm preserving homomorphism `NormedAddGroupHom α (Completion α)` from `NormedAddCommGroup.toCompl` to `UniformSpace.Completion.coeNormedAddGroupHom`. - We analogously rename some other theorems. - We add some trivial theorems (all of which are proved by `rfl`) that state that the functions considered above are equal. We give all of them the `simp` and `norm_cast` attributes. - We add a new theorem `UniformSpace.Completion.coeAddHom_eq_coe` that states that `UniformSpace.Completion.coeAddHom` and `UniformSpace.Completion.coe` are equal as functions. - We similarly add a new theorem `UniformSpace.Completion.coeRingHom_eq_coe`. - We rename the theorem `UniformSpace.Completion.coe_toComplₗᵢ` to `UniformSpace.Completion.coeₗᵢ_eq_coe`. - We rename the theorem `UniformSpace.Completion.coe_toComplL` to `UniformSpace.Completion.coeL_eq_coe`. - We similarly add a new theorem `UniformSpace.Completion.coeNormedAddGroupHom_eq_coe`. - We change all occurrences of the string `((↑) : α → Completion α)` to `(coe : α → Completion α)` or just `coe`. - We put the statements of some theorems into simp normal form by using the plain function `coe` rather than the homomorphisms that carry more structure. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology merge-conflict 130/92 Mathlib/Analysis/Analytic/Uniqueness.lean,Mathlib/Analysis/Calculus/FDeriv/Analytic.lean,Mathlib/Analysis/Complex/AbsMax.lean,Mathlib/Analysis/Complex/Liouville.lean,Mathlib/Analysis/InnerProductSpace/Completion.lean,Mathlib/Analysis/Normed/Group/HomCompletion.lean,Mathlib/Analysis/Normed/Module/Completion.lean,Mathlib/Analysis/SpecialFunctions/NonIntegrable.lean,Mathlib/MeasureTheory/Integral/IntegralEqImproper.lean,Mathlib/Topology/Algebra/GroupCompletion.lean,Mathlib/Topology/Algebra/InfiniteSum/GroupCompletion.lean,Mathlib/Topology/Algebra/InfiniteSum/Nonarchimedean.lean,Mathlib/Topology/Algebra/Nonarchimedean/Completion.lean,Mathlib/Topology/Algebra/UniformRing.lean,Mathlib/Topology/Category/UniformSpace.lean,Mathlib/Topology/MetricSpace/Completion.lean,Mathlib/Topology/UniformSpace/Completion.lean 17 4 ['eric-wieser', 'github-actions', 'trivial1711'] nobody
147-18579
4 months ago
147-18579
4 months ago
6-66637
6 days
17739 Aaron1011
author:Aaron1011
feat(Topology/Order/DenselyOrdered): prove Not (IsOpen) for intervals Prove that Iic/Ici/Ioc/Ico/Icc intervals are not open in densely ordered topologies with no min/max element --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-topology merge-conflict awaiting-author 27/0 Mathlib/Topology/Order/DenselyOrdered.lean 1 8 ['github-actions', 'vihdzp'] nobody
145-5854
4 months ago
145-5854
4 months ago
0-4704
1 hour
18474 FR-vdash-bot
author:FR-vdash-bot
perf: lower the priority of `*WithOne.to*` instances --- From #7873. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data slow-typeclass-synthesis t-algebra merge-conflict
label:t-algebra$
9/2 Mathlib/Algebra/Polynomial/BigOperators.lean,Mathlib/Data/Int/Cast/Defs.lean,Mathlib/Data/Nat/Cast/Defs.lean 3 7 ['FR-vdash-bot', 'eric-wieser', 'github-actions', 'leanprover-bot'] nobody
145-5609
4 months ago
145-5609
4 months ago
76-67978
76 days
20656 Komyyy
author:Komyyy
feat(Mathlib/Geometry/Manifold/VectorBundle/Sphere): convert orthogonal smooth `M → 𝕊ⁿ` & `M → ℝⁿ⁺¹` to smooth `M → T𝕊ⁿ` Current Mathlib has no easy way to define function from a manifold to tangent bundles of sphere: `T𝕊ⁿ`. This PR gives this: `sphereTangentMap`. This convert orthogonal smooth `M → 𝕊ⁿ` & `M → ℝⁿ⁺¹` to smooth `M → T𝕊ⁿ`. I also proved that if `f : M → 𝕊ⁿ` & `g : M → ℝⁿ⁺¹` are smooth then `sphereTangentMap` of `f` & `g` is smooth too. --- ⚠ **CAUTION** I formalized this in my spare time. I don't have the energy to maintain the PR, but I create this PR so this may helps everyone. The only one thing to do is proof cleanup. TODO: - [x] `contDiff_uncurry_stereoInvFunAux` & `coe_sphere_comp_stereoInvFun` may have to be moved to `Mathlib.Geometry.Manifold.Instances.Sphere`. - [ ] Proof cleanup. Current proof may be redundant and ugly. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-differential-geometry merge-conflict please-adopt 246/6 Mathlib.lean,Mathlib/Geometry/Manifold/Instances/Sphere.lean,Mathlib/Geometry/Manifold/VectorBundle/Sphere.lean 3 1 ['github-actions'] nobody
144-40543
4 months ago
144-40543
4 months ago
0-0
0 seconds
19596 Command-Master
author:Command-Master
feat(RingTheory/Valuation/PrimeMultiplicity): define `WithTop ℤ`-valued prime multiplicity on a fraction field Moves: - `multiplicity_addValuation` -> `AddValuation.multiplicity` - `multiplicity_addValuation_apply` -> `AddValuation.multiplicity_apply` --- - [x] depends on: #19149 - [x] depends on: #18786 - [x] depends on: #19122 - [x] depends on: #18954 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-algebra merge-conflict awaiting-author
label:t-algebra$
101/37 Mathlib/Data/ENat/Basic.lean,Mathlib/RingTheory/DiscreteValuationRing/Basic.lean,Mathlib/RingTheory/Valuation/PrimeMultiplicity.lean 3 11 ['ChrisHughes24', 'Command-Master', 'Vierkantor', 'faenuccio', 'github-actions', 'mathlib4-dependent-issues-bot'] nobody
144-30378
4 months ago
144-30378
4 months ago
8-2214
8 days
19091 Vierkantor
author:Vierkantor
chore(Algebra/MonoidAlgebra): split Defs.lean further This PR further splits the big file `MonoidAlgebra/Defs.lean` to focus on the ring structure on (`Add`)`MonoidAlgebra`. The following files have been split off: * `MonoidAlgebra/Lift.lean`: definition of `liftNC` * `MonoidAlgebra/MapDomain.lean`: definition of `mapDomain` * `MonoidAlgebra/Module.lean`: module structure (and some submodule results) * `MonoidAlgebra/Opposite.lean`: results on the `MulOpposite` ring structure I also changed one proof about scalar multiplication by natural numbers, so that it wouldn't need a full on module structure on `Finsupp`. This required adding a pair of lemmas on the definition of multiplying `Finsupp`s by natural numbers. --- - [ ] depends on: #19087 - [ ] depends on: #19205 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict
label:t-algebra$
883/560 Mathlib.lean,Mathlib/Algebra/MonoidAlgebra/Basic.lean,Mathlib/Algebra/MonoidAlgebra/Defs.lean,Mathlib/Algebra/MonoidAlgebra/Division.lean,Mathlib/Algebra/MonoidAlgebra/Lift.lean,Mathlib/Algebra/MonoidAlgebra/MapDomain.lean,Mathlib/Algebra/MonoidAlgebra/Module.lean,Mathlib/Algebra/MonoidAlgebra/Opposite.lean,Mathlib/Algebra/MonoidAlgebra/Support.lean,Mathlib/Algebra/Polynomial/Basic.lean,Mathlib/Data/Finsupp/Defs.lean,Mathlib/RingTheory/Polynomial/Opposites.lean 12 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
144-27126
4 months ago
144-27126
4 months ago
2-72196
2 days
15720 znssong
author:znssong
feat(SimpleGraph): The Bondy-Chvátal theorem The proof of the Bondy-Chvátal theorem, with Dirac's theorem and Ore's theorem as its corollary. - [x] depends on: #15536 - [ ] depends on: #15711 - [ ] depends on: #15578 new-contributor t-combinatorics merge-conflict blocked-by-other-PR 903/3 Mathlib.lean,Mathlib/Combinatorics/SimpleGraph/BondyChvatal.lean,Mathlib/Combinatorics/SimpleGraph/Finite.lean,Mathlib/Combinatorics/SimpleGraph/Hamiltonian.lean,Mathlib/Combinatorics/SimpleGraph/Path.lean,Mathlib/Combinatorics/SimpleGraph/Walk.lean,Mathlib/Dynamics/FixedPoints/Basic.lean,Mathlib/Dynamics/FixedPoints/Increasing.lean 8 3 ['github-actions', 'grunweg', 'leanprover-community-mathlib4-bot'] YaelDillies
assignee:YaelDillies
144-24940
4 months ago
144-24940
4 months ago
0-1791
29 minutes
15711 znssong
author:znssong
feat(Combinatorics/SimpleGraph): Some lemmas about walk, cycle and Hamiltonian cycle --- These lemmas are separated from the `meow-sister/BondyChvatal` branch and will be needed for the proof of the Bondy-Chvátal theorem. - [x] depends on: #15536 - [x] depends on: #16294 new-contributor t-combinatorics merge-conflict awaiting-author 407/3 Mathlib/Combinatorics/SimpleGraph/Finite.lean,Mathlib/Combinatorics/SimpleGraph/Hamiltonian.lean,Mathlib/Combinatorics/SimpleGraph/Path.lean,Mathlib/Combinatorics/SimpleGraph/Walk.lean 4 22 ['Rida-Hamadani', 'YaelDillies', 'github-actions', 'mathlib4-dependent-issues-bot', 'znssong'] nobody
144-24940
4 months ago
144-24940
4 months ago
9-13962
9 days
18629 tomaz1502
author:tomaz1502
feat(Computability.Timed): Formalization of runtime complexity of List.merge This PR adds the formalization of the runtime complexity of the merge function, defined in `Data/List/Sort`. Requires: https://github.com/leanprover-community/mathlib4/pull/15450 References: - Previous PR on mathlib3: https://github.com/leanprover-community/mathlib3/pull/14494/ - First discussion on Zulip: https://leanprover.zulipchat.com/#narrow/stream/113488-general/topic/BSc.20Final.20Project/near/220647062 - Second disussion on Zulip: https://leanprover.zulipchat.com/#narrow/stream/113488-general/topic/Formalization.20of.20Runtime.20Complexity.20of.20Sorting.20Algorithms/near/284184450 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-computability new-contributor merge-conflict awaiting-author 186/0 Mathlib.lean,Mathlib/Computability/Timed/InsertionSort.lean,Mathlib/Computability/Timed/Merge.lean 3 2 ['github-actions', 'trivial1711'] nobody
143-77259
4 months ago
143-77259
4 months ago
33-11262
33 days
17246 pechersky
author:pechersky
feat(RingTheory/PrimaryDecomposition): PIR of Noetherian under jacobson condition --- - [x] depends on: #17634 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict awaiting-author
label:t-algebra$
653/1 Mathlib.lean,Mathlib/NumberTheory/KummerDedekind.lean,Mathlib/RingTheory/Ideal/Maps.lean,Mathlib/RingTheory/Ideal/Operations.lean,Mathlib/RingTheory/Ideal/Quotient/Operations.lean,Mathlib/RingTheory/Jacobson/Ideal.lean,Mathlib/RingTheory/PrimaryDecomposition.lean,docs/references.bib 8 8 ['erdOne', 'github-actions', 'mathlib4-dependent-issues-bot'] erdOne
assignee:erdOne
143-33231
4 months ago
143-33231
4 months ago
13-7138
13 days
14412 jjaassoonn
author:jjaassoonn
feat: show stalk of presheaf of modules is a module over stalk of ring --- - [x] depends on: #14413 - [ ] depends on: #14501 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) workshop-AIM-AG-2024 t-algebraic-geometry merge-conflict blocked-by-other-PR 966/2 Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Presheaf/OverColimitsRing'.lean,Mathlib/Algebra/Category/ModuleCat/Presheaf/OverColimitsRing.lean,Mathlib/CategoryTheory/Filtered/Basic.lean,Mathlib/CategoryTheory/Limits/ConcreteCategory.lean,Mathlib/Geometry/RingedSpace/Basic.lean,Mathlib/Geometry/RingedSpace/Module.lean,Mathlib/Topology/Sheaves/Stalks.lean 8 5 ['github-actions', 'jjaassoonn', 'leanprover-community-mathlib4-bot', 'smorel394'] nobody
142-9442
4 months ago
298-33062
9 months ago
0-0
0 seconds
8362 urkud
author:urkud
feat(Asymptotics): define `ReflectsGrowth` --- - [x] depends on: #8349 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis merge-conflict awaiting-author 268/0 Mathlib.lean,Mathlib/Analysis/Asymptotics/ReflectsGrowth.lean 2 14 ['YaelDillies', 'fpvandoorn', 'github-actions', 'leanprover-community-mathlib4-bot', 'urkud'] nobody
141-84513
4 months ago
141-84513
4 months ago
1-41158
1 day
6692 prakol16
author:prakol16
feat: disjoint indexed union of local homeomorphisms Add disjoint indexed union of local equivs and local homeomorphisms --- This is leading up to PRing some things related to covering spaces that I wrote a long time ago in lean 3 but never submitted a PR for. Note that this was converted using mathport. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology merge-conflict awaiting-author 126/0 Mathlib/Logic/Equiv/PartialEquiv.lean,Mathlib/Topology/PartialHomeomorph.lean 2 4 ['alreadydone', 'github-actions', 'winstonyin'] nobody
141-69109
4 months ago
141-69109
4 months ago
117-22351
117 days
19291 PieterCuijpers
author:PieterCuijpers
feat(Algebra/Order/Hom): add quantale homomorphism Definition of quantale homomorphisms as functions that are both semigroup homomorphisms and complete lattice homomorphisms. --- - [x] depends on: #19810 - [x] depends on: #19811 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra merge-conflict awaiting-author
label:t-algebra$
209/0 Mathlib.lean,Mathlib/Algebra/Order/Hom/Quantale.lean,scripts/noshake.json 3 29 ['PieterCuijpers', 'YaelDillies', 'github-actions', 'kim-em', 'mathlib4-dependent-issues-bot'] nobody
139-12518
4 months ago
139-12519
4 months ago
36-2255
36 days
19352 hrmacbeth
author:hrmacbeth
chore: change some `nlinarith`s to `linear_combination`s --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP 13/13 Archive/Imo/Imo2021Q1.lean,Archive/Wiedijk100Theorems/AreaOfACircle.lean,Mathlib/Analysis/Normed/Group/AddCircle.lean,Mathlib/Analysis/Normed/Group/Basic.lean,Mathlib/Analysis/Normed/Ring/Units.lean,Mathlib/Analysis/SpecialFunctions/Complex/LogBounds.lean,Mathlib/Combinatorics/SimpleGraph/Regularity/Increment.lean,Mathlib/NumberTheory/Modular.lean 8 4 ['github-actions', 'hrmacbeth', 'leanprover-bot'] nobody
137-41729
4 months ago
137-41729
4 months ago
0-8636
2 hours
20477 artie2000
author:artie2000
feat(Aesop): Improve SetLike ruleset * Make many safe Aesop rules in the SetLike ruleset either unsafe or (additionally) simp lemmas * Add new Aesop rules `.closure_mem_of_mem` and `mem_of_star_mem` * Replace `simps` auto-generated lemmas around `StarAlgebra.adjoin` with an Aesop-registered API * Add new library note [SetLike Aesop ruleset] explaining the principles behind the new design The `simps` auto-generated lemmas I have removed produced messy output that harmed the performance of simp and Aesop without being particularly usable. The new API brings `StarAlgebra.adjoin` and friends in line with anlogous operations elsewhere in Mathlib. Moves (incidental): `NonUnitalSubalgebra.starClosure_toNonunitalSubalgebra` -> `NonUnitalSubalgebra.starClosure_toNonUnitalSubalgebra` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-meta merge-conflict awaiting-author
label:t-algebra$
201/85 Mathlib/Algebra/Algebra/NonUnitalSubalgebra.lean,Mathlib/Algebra/Algebra/Subalgebra/Basic.lean,Mathlib/Algebra/Field/Subfield/Basic.lean,Mathlib/Algebra/Field/Subfield/Defs.lean,Mathlib/Algebra/Group/Subgroup/Basic.lean,Mathlib/Algebra/Group/Subgroup/Defs.lean,Mathlib/Algebra/Group/Subgroup/Lattice.lean,Mathlib/Algebra/Group/Submonoid/Basic.lean,Mathlib/Algebra/Group/Submonoid/Defs.lean,Mathlib/Algebra/Group/Submonoid/Pointwise.lean,Mathlib/Algebra/Group/Subsemigroup/Basic.lean,Mathlib/Algebra/Group/Subsemigroup/Defs.lean,Mathlib/Algebra/Lie/Subalgebra.lean,Mathlib/Algebra/Lie/Submodule.lean,Mathlib/Algebra/Module/Bimodule.lean,Mathlib/Algebra/Module/Submodule/Defs.lean,Mathlib/Algebra/Module/Submodule/Lattice.lean,Mathlib/Algebra/Order/Ring/Cone.lean,Mathlib/Algebra/Order/Star/Basic.lean,Mathlib/Algebra/Polynomial/Module/AEval.lean,Mathlib/Algebra/Ring/Subring/Basic.lean,Mathlib/Algebra/Ring/Subring/Defs.lean,Mathlib/Algebra/Ring/Subsemiring/Basic.lean,Mathlib/Algebra/Ring/Subsemiring/Defs.lean,Mathlib/Algebra/Star/Basic.lean,Mathlib/Algebra/Star/NonUnitalSubalgebra.lean,Mathlib/Algebra/Star/SelfAdjoint.lean,Mathlib/Algebra/Star/Subalgebra.lean,Mathlib/Analysis/Convex/Cone/Basic.lean,Mathlib/Data/SetLike/Basic.lean,Mathlib/FieldTheory/IntermediateField/Basic.lean,Mathlib/GroupTheory/GroupAction/SubMulAction.lean,Mathlib/LinearAlgebra/RootSystem/WeylGroup.lean,Mathlib/LinearAlgebra/Span/Defs.lean,Mathlib/MeasureTheory/Function/StronglyMeasurable/Basic.lean,Mathlib/MeasureTheory/Measure/MeasureSpaceDef.lean,Mathlib/NumberTheory/KummerDedekind.lean,Mathlib/Order/BooleanSubalgebra.lean,Mathlib/RingTheory/Adjoin/Basic.lean,Mathlib/RingTheory/DedekindDomain/Different.lean,Mathlib/RingTheory/EssentialFiniteness.lean,Mathlib/RingTheory/GradedAlgebra/HomogeneousLocalization.lean,Mathlib/RingTheory/NonUnitalSubring/Basic.lean,Mathlib/RingTheory/NonUnitalSubsemiring/Basic.lean,Mathlib/RingTheory/TwoSidedIdeal/Basic.lean,Mathlib/Tactic/SetLike.lean,Mathlib/Topology/Algebra/Algebra.lean,Mathlib/Topology/Algebra/NonUnitalAlgebra.lean,Mathlib/Topology/Algebra/NonUnitalStarAlgebra.lean,Mathlib/Topology/Algebra/StarSubalgebra.lean 50 62 ['JLimperg', 'YaelDillies', 'artie2000', 'github-actions', 'leanprover-bot', 'madvorak'] nobody
135-34899
4 months ago
135-34899
4 months ago
14-64862
14 days
20836 artie2000
author:artie2000
refactor: Abstract out the substructure lattice construction and SetLike closure operators --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict 354/175 Mathlib/Algebra/Group/Subsemigroup/Basic.lean,Mathlib/Algebra/Group/Subsemigroup/Defs.lean,Mathlib/Data/SetLike/Basic.lean,Mathlib/Data/SetLike/Closure.lean,Mathlib/Order/CompleteLattice.lean 5 2 ['artie2000', 'github-actions'] nobody
133-18703
4 months ago
133-18703
4 months ago
0-0
0 seconds
20372 jvlmdr
author:jvlmdr
feat(MeasureTheory/Function): Add ContinuousLinearMap.bilinearCompLp(L) Introduce ContinuousLinearMap.bilinearCompLp and bilinearCompLpL. Generalize eLpNorm_le_eLpNorm_mul_eLpNorm theorems to include constant C in bound condition. --- Expect this may be useful for defining tempered distributions from functions in `L^p`. The definitions more or less follow `ContinuousLinearMap.compLp...`. Names are loosely analogous to `ContinuousLinearMap.bilinearComp` and `SchwartzMap.bilinLeftCLM`. Note: I preferred the spelling `hpqr : p⁻¹ + q⁻¹ = r⁻¹` with `f` in `L^p` and `g` in `L^q` to `hpqr : 1 / p = 1 / q + 1 / r`. It's easier to obtain from `ENNReal.IsConjExponent` too. A few questions: - [ ] I defined `bilinear{Left,Right}LpL` in addition to `bilinearCompLpL` because `LinearMap.mkContinuous₂` is marked as `noncomputable` and `LinearMap.mkContinuous` is not. Is this worth the extra definitions? (Note: This is not visible in the source due to `noncomputable section`.) - [ ] Should I use `C : ℝ` instead of `C : NNReal` for `eLpNorm_le_eLpNorm_mul_eLpNorm'_of_norm'`? - [ ] Is it going to be painful to have `[Fact (1 ≤ p)] [Fact (1 ≤ q)] [Fact (1 ≤ r)]`? I don't think there's a way to avoid it though. Maybe providing specialized versions for `p.IsConjExponent q` with `L^1`? Naming: - [ ] Is it satisfactory to add a `'` to the `eLpNorm_le_eLpNorm_mul_eLpNorm ` definitions in `CompareExp.lean` where `≤ ‖f x‖ * ‖g x‖` has been replaced with `≤ C * ‖f x‖ * ‖g x‖`? These could replace the existing theorems, although I don't want to break backwards compatibility. There are 5 instances: `eLpNorm_le_eLpNorm_top_mul_eLpNorm'`, `eLpNorm_le_eLpNorm_mul_eLpNorm_top'`, `eLpNorm'_le_eLpNorm'_mul_eLpNorm''`, `eLpNorm_le_eLpNorm_mul_eLpNorm_of_nnnorm'`, `eLpNorm_le_eLpNorm_mul_eLpNorm'_of_norm'` (I'm not sure why the existing theorem `eLpNorm_le_eLpNorm_mul_eLpNorm'_of_norm` has an internal `'`) - [ ] Is `bilinearLeftLpL` a suitable name? Other options: `bilinearCompLpLeftL`, `bilinearCompLeftLpL`, `bilinLeftLpL` (analogous to `SchwartzMap.bilinLeftCLM`) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-measure-probability merge-conflict 203/40 Mathlib/MeasureTheory/Function/LpSeminorm/CompareExp.lean,Mathlib/MeasureTheory/Function/LpSpace.lean 2 1 ['github-actions'] nobody
132-29866
4 months ago
132-29866
4 months ago
27-43617
27 days
17176 arulandu
author:arulandu
feat: integrals and integrability with .re Lemmas for swapping order of .re and integration/integrability. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-measure-probability merge-conflict awaiting-author 49/0 Mathlib/MeasureTheory/Function/L1Space.lean,Mathlib/MeasureTheory/Integral/IntegrableOn.lean,Mathlib/MeasureTheory/Integral/IntervalIntegral.lean,Mathlib/MeasureTheory/Integral/SetIntegral.lean 4 30 ['EtienneC30', 'arulandu', 'github-actions', 'loefflerd'] nobody
131-4299
4 months ago
131-4299
4 months ago
9-73631
9 days
20872 grunweg
author:grunweg
feat: lint against the tactic.skipAssignedInstances option in mathlib This means we can remove the corresponding technical debt entry. We also correct some outdated details in the Linter/Style.lean docstring. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) tech debt t-linter merge-conflict awaiting-author 63/7 Mathlib/Analysis/InnerProductSpace/PiL2.lean,Mathlib/Tactic/Linter/Style.lean,Mathlib/Topology/Separation/Regular.lean,MathlibTest/LintStyle.lean,scripts/technical-debt-metrics.sh 5 17 ['adomani', 'github-actions', 'grunweg'] nobody
130-84729
4 months ago
130-84729
4 months ago
0-9411
2 hours
2605 eric-wieser
author:eric-wieser
chore: better error message in linarith On this mwe: ```lean import Mathlib.Tactic.Linarith example (s : Set ℕ) (h : s = s) : 0 ≤ 1 := by linarith ``` this now indicates where the internal error is coming from. Is there a better way of chaining errors than this? --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta merge-conflict awaiting-author 12/1 Mathlib/Tactic/Linarith/Preprocessing.lean 1 3 ['Vierkantor', 'harahu', 'kim-em', 'mo271'] nobody
130-20459
4 months ago
564-80146
1 year ago
4-7271
4 days
3171 eric-wieser
author:eric-wieser
refactor: make the algebra hierarchy use flat structures By introducing a `FlatHack` base class and using it as the first parent of every algebra typeclass, it causes the typeclasses to all overlap and so we emulate flat structures. Most of the pain here comes from `to_additive` not generating any of the ancestor projections properly; this was already a bug present for `n + 1` parents, but now the `1` is taken up This is one workaround for leanprover/lean4#2074: don't let the eta-diamonds appear in the first place. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP 328/240 .github/workflows/build.yml,Mathlib/Algebra/Algebra/Equiv.lean,Mathlib/Algebra/Algebra/Hom.lean,Mathlib/Algebra/Category/GroupCat/Basic.lean,Mathlib/Algebra/Category/GroupCat/EquivalenceGroupAddGroup.lean,Mathlib/Algebra/Category/MonCat/FilteredColimits.lean,Mathlib/Algebra/DualNumber.lean,Mathlib/Algebra/Field/Defs.lean,Mathlib/Algebra/GCDMonoid/Basic.lean,Mathlib/Algebra/Group/Basic.lean,Mathlib/Algebra/Group/Defs.lean,Mathlib/Algebra/Group/Ext.lean,Mathlib/Algebra/Group/Opposite.lean,Mathlib/Algebra/Group/Prod.lean,Mathlib/Algebra/GroupPower/Lemmas.lean,Mathlib/Algebra/Hom/Group.lean,Mathlib/Algebra/MonoidAlgebra/Basic.lean,Mathlib/Algebra/Order/Chebyshev.lean,Mathlib/Algebra/Order/Group/Abs.lean,Mathlib/Algebra/Order/Group/Defs.lean,Mathlib/Algebra/Order/Module.lean,Mathlib/Algebra/Order/Rearrangement.lean,Mathlib/Algebra/Order/Ring/Canonical.lean,Mathlib/Algebra/Order/Ring/Defs.lean,Mathlib/Algebra/Quandle.lean,Mathlib/Algebra/Ring/Defs.lean,Mathlib/Algebra/TrivSqZeroExt.lean,Mathlib/CategoryTheory/Endomorphism.lean,Mathlib/CategoryTheory/Preadditive/Basic.lean,Mathlib/CategoryTheory/Preadditive/SingleObj.lean,Mathlib/Data/Finsupp/Multiset.lean,Mathlib/Data/Int/LeastGreatest.lean,Mathlib/Data/Int/Order/Basic.lean,Mathlib/Data/Int/Order/Lemmas.lean,Mathlib/Data/Nat/Choose/Multinomial.lean,Mathlib/Data/Real/CauSeqCompletion.lean,Mathlib/Data/ZMod/Defs.lean,Mathlib/LinearAlgebra/AffineSpace/Ordered.lean,Mathlib/LinearAlgebra/LinearPMap.lean,Mathlib/RingTheory/Ideal/Quotient.lean,Mathlib/Tactic/Positivity/Core.lean,Mathlib/Tactic/Ring/Basic.lean 42 14 ['eric-wieser', 'gebner', 'harahu'] nobody
130-20444
4 months ago
678-28652
1 year ago
0-0
0 seconds
11837 trivial1711
author:trivial1711
feat: completion of a uniform multiplicative group Multiplicativize `Topology.Algebra.GroupCompletion`. That is, rewrite it in the multiplicative setting and recover the original results using `@[to_additive]`. - Because `@[to_additive]` doesn't work with `noncomputable section` (https://github.com/leanprover/lean4/pull/2610), some instances with `@[to_additive]` need to be explicitly marked with `noncomputable instance`. - One might be tempted to multiplicativize this definition from `Topology.Algebra.GroupCompletion`: ```lean instance [UniformSpace α] [Add α] : Add (Completion α) := ⟨Completion.map₂ (· + ·)⟩ ``` to this: ```lean @[to_additive] instance [UniformSpace α] [Mul α] : Mul (Completion α) := ⟨Completion.map₂ (· * ·)⟩ ``` However, as Eric Wieser pointed out, doing so would create a bad diamond with the definition ```lean instance [UniformSpace α] [TopologicalRing α] [UniformAddGroup α] [Ring α] : Mul (Completion α) := ⟨curry <| (denseInducing_coe.prod denseInducing_coe).extend ((↑) ∘ uncurry (· * ·))⟩ ``` in `Topology.Algebra.UniformRing`. How should this diamond be resolved? Well, the definition of multiplication that uses `curry <| (denseInducing_coe.prod denseInducing_coe).extend ((↑) ∘ uncurry (· * ·))` is the "correct" one. For example, it yields the correct result if `α` is `ℚ`, unlike the definition that uses `Completion.map₂ (· * ·)`. (This is because `Completion.map₂` yields junk values if used on a function which is not uniformly continuous. Note, however, that if multiplication on `α` *is* uniformly continuous, then `Completion.map₂ (· * ·)` and `curry <| (denseInducing_coe.prod denseInducing_coe).extend ((↑) ∘ uncurry (· * ·))` are propositionally equal.) So, following Eric's suggestion, we remove the definition that uses `Completion.map₂ (· * ·)`, and generalize the other definition to any uniform space with a multiplication operation: ```lean @[to_additive] noncomputable instance [UniformSpace α] [Mul α] : Mul (Completion α) := ⟨curry <| (denseInducing_coe.prod denseInducing_coe).extend ((↑) ∘ uncurry (· * ·))⟩ ``` This requires slightly modifying some of the proofs in `Topology.Algebra.GroupCompletion`. For example, suppose that `α` is a uniform group. Since we can no longer use `Completion.continuous_map₂`, it becomes more efficient to prove that the multiplication, inversion, and division operations on `Completion α` are uniformly continuous *before* we prove that `Completion α` is a group. - Previously, `Topology.Algebra.GroupCompletion` had an instance: ```lean instance [UniformSpace α] [Sub α] : Sub (Completion α) := ... ``` Naively multiplicativizing this would yield ```lean @[to_additive] instance [UniformSpace α] [Inv α] : Inv (Completion α) := ... ``` Unfortunately, this would conflict with `Topology.Algebra.UniformField`, which already instantiates `Inv (Completion α)` when `α` is a uniform field. Instead, we use two different `instance` declarations. (If `α` is an additive group, then this instantiates `Neg (Completion α)` twice, and the instances are syntactically equal.) ```lean @[to_additive] noncomputable instance [UniformSpace α] [Group α] : Inv (Completion α) := ... instance [UniformSpace α] [Neg α] : Neg (Completion α) := ... ``` This avoids the bad diamond (because a uniform field can never be a `Group`) while remaining backward compatible. Note that the `@[to_additive]` is necessary here, because it maintains the link between the additive setting and multiplicative setting. We use a similar method to instantiate `Div (Completion α)`. - Some definitions in this file involve a module structure on `α`. We leave these as is and do not attempt to multiplicativize them at all. - The instance of `DistribMulAction` must be multiplicativized to an instance of `MulDistribMulAction` manually. Zulip thread: https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/Completion.20of.20a.20uniform.20multiplicative.20group --- # (Small) Issue Recall the following trick that this pull request uses to define inversion and negation on uniform spaces. The idea is that we define negation on the completion of any uniform space that has a negation operation, but we define inversion on only the completion of a uniform space that has the structure of a multiplicative group. We do this to avoid creating a bad diamond with the inversion operation on a uniform field. ```lean @[to_additive] noncomputable instance {α : Type*} [UniformSpace α] [Group α] : Inv (Completion α) := ... instance {α : Type*} [UniformSpace α] [Neg α] : Neg (Completion α) := ... ``` Now, suppose that we want to prove `coe_inv_of_group` (resp. `coe_neg`), which states that the coercion `α → Completion α` commutes with inversion (resp. negation). In the current version of this pull request, `coe_inv_of_group` (resp. `coe_neg`) only applies to uniform multiplicative (resp. additive) groups. However, we do not use the fact that multiplication (resp. addition) on `α` is uniformly continuous to prove it. We only use the fact that inversion (resp. negation) is continuous. So, what we really want is to have more general statements that look like this: ```lean theorem coe_inv_of_group {α : Type*} [UniformSpace α] [Group α] [ContinuousInv α] : ... theorem coe_neg {α : Type*} [UniformSpace α] [Neg α] [ContinuousNeg α] : ... ``` Note that `coe_inv_of_group` needs the assumption `[Group α]`, because otherwise inversion is not defined on `Completion α` at all. However, `coe_neg` does not need the analogous assumption `[AdditiveGroup α]`. The question is: If `coe_inv_of_group` and `coe_neg` are written in this more general form, how can we link them using `@[to_additive]`? Here is one option, but it obviously leaves something to be desired. ```lean @[to_additive coe_neg_do_not_use_this_use_the_more_general_version] theorem coe_inv_of_group {α : Type*} [UniformSpace α] [Group α] [ContinuousInv α] : ... theorem coe_neg {α : Type*} [UniformSpace α] [Neg α] [ContinuousNeg α] : ... ``` Co-authored-by: Eric Wieser --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-topology merge-conflict WIP help-wanted
label:t-algebra$
342/217 Mathlib/Analysis/InnerProductSpace/Completion.lean,Mathlib/Analysis/Normed/Group/HomCompletion.lean,Mathlib/Analysis/Normed/Module/Completion.lean,Mathlib/Topology/Algebra/GroupCompletion.lean,Mathlib/Topology/Algebra/InfiniteSum/GroupCompletion.lean,Mathlib/Topology/Algebra/Nonarchimedean/Completion.lean,Mathlib/Topology/Algebra/UniformField.lean,Mathlib/Topology/Algebra/UniformMulAction.lean,Mathlib/Topology/Algebra/UniformRing.lean 9 14 ['eric-wieser', 'github-actions', 'trivial1711'] nobody
129-84364
4 months ago
129-84364
4 months ago
101-64856
101 days
12670 trivial1711
author:trivial1711
feat: completion of a nonarchimedean multiplicative group We prove that the completion of a nonarchimedean multiplicative group is a nonarchimedean multiplicative group. --- - [x] depends on: #12669 - [ ] depends on: #11837 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-topology merge-conflict blocked-by-other-PR
label:t-algebra$
358/228 Mathlib/Analysis/InnerProductSpace/Completion.lean,Mathlib/Analysis/Normed/Group/HomCompletion.lean,Mathlib/Analysis/Normed/Module/Completion.lean,Mathlib/Topology/Algebra/GroupCompletion.lean,Mathlib/Topology/Algebra/InfiniteSum/GroupCompletion.lean,Mathlib/Topology/Algebra/Nonarchimedean/Completion.lean,Mathlib/Topology/Algebra/UniformField.lean,Mathlib/Topology/Algebra/UniformMulAction.lean,Mathlib/Topology/Algebra/UniformRing.lean 9 n/a ['github-actions', 'leanprover-community-mathlib4-bot'] nobody
129-84241
4 months ago
unknown
unknown
14799 luigi-massacci
author:luigi-massacci
feat(Analysis/MeanInequalities): Weighted QM-AM inequality The inequality between the quadratic and arithmetic mean as a consequence of Jensen's inequality. Weighted version for positive real valued functions from a `Finset`. Fix notation for sums, switching to `∈` in place of `in`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-analysis easy merge-conflict awaiting-author 26/3 Mathlib/Analysis/MeanInequalities.lean 1 8 ['YaelDillies', 'acmepjz', 'github-actions', 'luigi-massacci', 'vihdzp'] nobody
129-83870
4 months ago
129-83870
4 months ago
0-38862
10 hours
12294 AntoineChambert-Loir
author:AntoineChambert-Loir
feat(Mathlib.RingTheory.TensorProduct.Polynomial) : tensor product of a (univariate) polynomial ring We define a linear equivalence of a polynomial ring by a module with a finsupp type. We prove lemmas that allow to manipulate this equivalence. This is adapted from the content of #12293, but since `Polynomial` is a structure containing a `Finsupp`, these functions can't be applied directly to `Polynomial`. Some linear equivs need to be added to mathlib for that. --- - [x] depends on: #12293 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict WIP
label:t-algebra$
484/0 Mathlib.lean,Mathlib/Algebra/MvPolynomial/Basic.lean,Mathlib/Algebra/Polynomial/Basic.lean,Mathlib/Data/Finsupp/Defs.lean,Mathlib/LinearAlgebra/TensorProduct/Tower.lean,Mathlib/RingTheory/TensorProduct/MvPolynomial.lean,Mathlib/RingTheory/TensorProduct/Polynomial.lean 7 1 ['leanprover-community-mathlib4-bot'] nobody
129-30189
4 months ago
129-30189
4 months ago
0-79429
22 hours
18438 ADedecker
author:ADedecker
refactor: adapt `KrullTopology` to the new algebraic filter bases API --- - [ ] depends on: #18437 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-topology merge-conflict blocked-by-other-PR
label:t-algebra$
771/168 Mathlib.lean,Mathlib/FieldTheory/KrullTopology.lean,Mathlib/Topology/Algebra/FilterBasis.lean,Mathlib/Topology/Algebra/FilterBasisNew.lean,Mathlib/Topology/Algebra/Nonarchimedean/Bases.lean,Mathlib/Topology/Algebra/Nonarchimedean/BasesNew.lean 6 5 ['ADedecker', 'AntoineChambert-Loir', 'github-actions', 'mathlib4-dependent-issues-bot'] nobody
129-822
4 months ago
129-822
4 months ago
0-638
10 minutes
12824 BoltonBailey
author:BoltonBailey
refactor: `ReflTransGen` It would be nice to have that `ReflTransGen` is the composition of `ReflGen` with `TransGen`, currently experimenting with redefining it this way. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-logic merge-conflict WIP help-wanted 91/96 Mathlib/Logic/Relation.lean 1 4 ['BoltonBailey', 'grunweg', 'vihdzp'] nobody
128-69017
4 months ago
130-82116
4 months ago
0-0
0 seconds
19890 vihdzp
author:vihdzp
chore(SetTheory/Ordinal/Arithmetic): redefine subtraction We redefine ordinal subtraction so as to make `add_sub_cancel_of_le` an immediate corollary. This ultimately allows us to give a much simpler proof for `add_le_of_limit` (now `add_le_iff_of_isLimit`). --- - [ ] depends on: #18893 - [x] depends on: #19888 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-set-theory merge-conflict blocked-by-other-PR 134/94 Mathlib/Order/InitialSeg.lean,Mathlib/Order/RelIso/Basic.lean,Mathlib/Order/RelIso/Set.lean,Mathlib/SetTheory/Ordinal/Arithmetic.lean,Mathlib/SetTheory/Ordinal/Basic.lean,Mathlib/SetTheory/Ordinal/FixedPoint.lean 6 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
128-37457
4 months ago
128-37457
4 months ago
0-155
2 minutes
14686 smorel394
author:smorel394
feat (AlgebraicGeometry/Grassmannian): define the Grassmannian scheme # The Grassmannian scheme Define the Grassmannian scheme by gluing affine charts. We fix a commutative ring `K`, a free `K`-module of finite type `V` and two natural numbers `r` and `c`. The scheme we define should parametrize surjective `K`-linear maps `V →ₗ[K] (Fin r → K)`, assuming that `V` is of rank `r + c`. We actually define the scheme without assuming the condition on the rank of `V`, but it is empty unless the rank of `V` is `r + c`. Main definitions: * `Grassmannian.glueData K V r c`: the `AlgebraicGeometry.Scheme.GlueData` defining the Grassmannian scheme. * `Grassmannian K V r c`: the Grassmannian scheme, defined as `(Grassmannian.glueData K V r c).glued`. * `Grassmannian.structMorphism K V r c`: the structural morphism from `Grassmannian K V r c` to `Spec K`. # Implementation We use as index type for the charts the type `Basis (Fin (r + c)) K V` (so this is empty unless `V` is free of rank `r + c`). All the charts are the same and equal to the affine space with coordinates indexed by `Fin c × Fin r`, that is, to `Spec (MvPolynomial (Fin c × Fin r) K)`. The idea is that, for `i` in `Basis (Fin (r + c)) K V`, the corresponding chart will parametrize all surjective `K`-linear maps `φ : V →ₗ[K] (Fin r → K)` that become isomorphisms when restricted to the `K`-submodule generated by the first `r` vectors of the basis `i`. To get the point of the chart corresponding to `φ`, we take the matrix of `φ` in the basis `i` of `V` and the canonical basis of `Fin r → K`, we divide it on the right by its top `r × r` square submatrix (which is invertible by assumption), and we taken the botton `c × r` submatrix. This is almost the usual description of the Grassmannian by charts, with three differences: * We consider the Grassmannian parametrizing `r`-dimensional quotients of `V` instead of `r`-dimensional subspaces of `V`, because this is more natural when working over a general ring (or scheme). * In the usual description, we fix a basis of `V` and index the chart by its subsets `I` of cardinality `r`. Here, to avoid making a choice, we instead index charts by the set of bases of `V` and always choose the subset `I` to consist of the first `r` vectors. * Instead of working with `FiniteDimensional.finrank K V - r`, which would cause technical trouble because of the way subtraction works on `ℕ`, we introduce the codimension `c` as an auxiliary variable, and our constructions are only interesting when `r + c` is equal to `FiniteDimensional.finrank K V`. # Why is this a WIP * There a bunch of lemmas in the file `AlgebraicGeometry/Grassmannian/Lemmas.lean` that either should not be necessary or should be put in another PR for some other part of mathlib. * The proofs in `AlgebraicGeometry/Grassmannian/Basic.lean` are probably too complicated, and the names suck. # Notes. This contribution was created as part of the AIM workshop "Formalizing algebraic geometry" in June 2024. --- - [x] depends on: #14711 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) workshop-AIM-AG-2024 t-algebraic-geometry merge-conflict please-adopt WIP 1002/0 Mathlib.lean,Mathlib/AlgebraicGeometry/Grassmannian/Basic.lean,Mathlib/AlgebraicGeometry/Grassmannian/Lemmas.lean 3 15 ['erdOne', 'github-actions', 'joelriou', 'leanprover-community-mathlib4-bot', 'smorel394'] nobody
125-44790
4 months ago
125-44790
4 months ago
0-201
3 minutes
9449 hmonroe
author:hmonroe
feat: Add Turing machine with the quintet definition (TMQ) and a chainable step function for each TM type --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-computability merge-conflict awaiting-author 458/1 Mathlib/Computability/TuringMachine.lean,Mathlib/Logic/PartArith.lean 2 8 ['eric-wieser', 'github-actions', 'hmonroe'] nobody
124-49043
4 months ago
124-49043
4 months ago
14-19968
14 days
18719 FR-vdash-bot
author:FR-vdash-bot
perf: lower the priority of `SemilinearMapClass.toAddHomClass` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-bench slow-typeclass-synthesis t-algebra merge-conflict
label:t-algebra$
14/7 Mathlib/Algebra/Module/LinearMap/Defs.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Unique.lean,MathlibTest/TCSynth.lean 3 4 ['FR-vdash-bot', 'github-actions', 'leanprover-bot'] nobody
123-23860
4 months ago
123-23860
4 months ago
0-0
0 seconds
20663 EtienneC30
author:EtienneC30
feat: `PFunLike` typeclass for partial homomorphisms and `LinearPMapClass` A test PR implementing a typeclass `PFunLike` to represent partial homomorphisms and building a `LinearPMapClass` typeclass. Started from [this](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/ContinuousLinearPMap) discussion. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data t-algebra merge-conflict WIP
label:t-algebra$
278/49 Mathlib.lean,Mathlib/Algebra/Group/PHom.lean,Mathlib/Algebra/Module/Injective.lean,Mathlib/Analysis/Convex/Cone/Extension.lean,Mathlib/Data/PFunLike.lean,Mathlib/GroupTheory/GroupAction/PHom.lean,Mathlib/LinearAlgebra/LinearPMap.lean 7 1 ['github-actions'] nobody
122-16308
4 months ago
122-16308
4 months ago
0-0
0 seconds
21474 erdOne
author:erdOne
feat(RingTheory): replace `Ring.DimensionLEOne` with `Ring.KrullDimLE` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-algebra merge-conflict
label:t-algebra$
285/170 Mathlib.lean,Mathlib/RingTheory/DedekindDomain/Basic.lean,Mathlib/RingTheory/DedekindDomain/Dvr.lean,Mathlib/RingTheory/DedekindDomain/Ideal.lean,Mathlib/RingTheory/DiscreteValuationRing/TFAE.lean,Mathlib/RingTheory/Ideal/Over.lean,Mathlib/RingTheory/KrullDimension/Basic.lean,Mathlib/RingTheory/KrullDimension/Localization.lean,Mathlib/RingTheory/KrullDimension/Polynomial.lean,Mathlib/RingTheory/KrullDimension/Quotient.lean,Mathlib/RingTheory/LocalRing/ResidueField/Basic.lean,Mathlib/RingTheory/Nilpotent/End.lean,Mathlib/RingTheory/Nilpotent/Lemmas.lean,Mathlib/RingTheory/PID/Quotient.lean,Mathlib/RingTheory/PrincipalIdealDomain.lean,Mathlib/RingTheory/Spectrum/Maximal/Localization.lean 16 1 ['github-actions'] nobody
122-10354
4 months ago
122-10354
4 months ago
2-7106
2 days
19697 quangvdao
author:quangvdao
feat(BigOperators/Fin): Sum/product over `Fin` intervals This PR adds new theorems about the sum/product of some vector over `Fin` intervals. One example is: ``` @[to_additive] theorem prod_Iic_succ (i : Fin n) : ∏ j ∈ Iic i.succ, v j = (∏ j ∈ Iic i.castSucc, v j) * v i.succ ``` --- - [x] depends on: #20360 This is in preparation for reworking `finSigmaFinEquiv` and `finProdFinEquiv` in #19013. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data merge-conflict awaiting-author 87/12 Mathlib/Algebra/BigOperators/Fin.lean,Mathlib/Data/Fintype/Fin.lean,Mathlib/Order/Interval/Finset/Fin.lean 3 20 ['Ruben-VandeVelde', 'YaelDillies', 'eric-wieser', 'github-actions', 'mathlib4-dependent-issues-bot', 'quangvdao'] nobody
122-5061
4 months ago
122-5061
4 months ago
6-25961
6 days
19353 hrmacbeth
author:hrmacbeth
chore: golf some term/rw proofs using `linear_combination` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP 47/102 Archive/Wiedijk100Theorems/SumOfPrimeReciprocalsDiverges.lean,Mathlib/Analysis/Convex/Slope.lean,Mathlib/Analysis/Seminorm.lean,Mathlib/MeasureTheory/Integral/RieszMarkovKakutani.lean,Mathlib/NumberTheory/Modular.lean,Mathlib/NumberTheory/Zsqrtd/Basic.lean,Mathlib/Topology/ContinuousMap/ZeroAtInfty.lean 7 5 ['github-actions', 'grunweg', 'hrmacbeth', 'leanprover-bot'] grunweg
assignee:grunweg
121-4182
4 months ago
121-4182
4 months ago
0-7781
2 hours
21196 vihdzp
author:vihdzp
chore: make argument of `zero_le` implicit This simplifies our expressions probably 95% of the time, and the remaining 5% we can simply use the Lean 4 implicit argument notation. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order awaiting-CI merge-conflict 10/10 Mathlib/Algebra/Order/Monoid/Canonical/Defs.lean 1 1 ['github-actions'] nobody
120-66704
4 months ago
120-66704
4 months ago
0-0
0 seconds
20248 peabrainiac
author:peabrainiac
feat(Topology/Compactness): first-countable locally path-connected spaces are delta-generated Shows that all first-countable locally path-connected spaces are delta-generated (so in particular all normed spaces and convex subsets thereof are), and that delta-generated spaces are equivalently generated by the unit interval or standard simplices. --- - [ ] depends on: #21616 In principle, this should be close to all that's required to show that all simplicial complexes and CW-complexes are delta-generated; I just haven't done it yet because I'm not sure which file to best do it in. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import new-contributor t-topology merge-conflict awaiting-author blocked-by-other-PR 1189/813 Mathlib.lean,Mathlib/Geometry/Manifold/ChartedSpace.lean,Mathlib/Topology/Algebra/Module/LocallyConvex.lean,Mathlib/Topology/Compactness/DeltaGeneratedSpace.lean,Mathlib/Topology/Connected/LocPathConnected.lean,Mathlib/Topology/Connected/PathConnected.lean,Mathlib/Topology/ContinuousOn.lean,Mathlib/Topology/Homotopy/HSpaces.lean,Mathlib/Topology/Path.lean 9 22 ['YaelDillies', 'github-actions', 'kbuzzard', 'mathlib4-dependent-issues-bot', 'peabrainiac'] nobody
119-73576
3 months ago
119-73576
3 months ago
39-21495
39 days
21610 JLimperg
author:JLimperg
Aesop forward benchmark: forward precomp Not a real PR, just for benchmarking. merge-conflict 30/27 Mathlib/Data/List/InsertIdx.lean,Mathlib/Tactic/Recall.lean,Mathlib/Topology/List.lean,Test.lean,lake-manifest.json,lakefile.lean,lean-toolchain 7 3 ['JLimperg', 'github-actions', 'leanprover-bot'] nobody
119-23067
3 months ago
120-11430
4 months ago*
0-0
0 seconds*
21611 JLimperg
author:JLimperg
Aesop forward benchmark: master no-precomp Not a real PR, just for benchmarking. merge-conflict 30/27 Mathlib/Data/List/InsertIdx.lean,Mathlib/Tactic/Recall.lean,Mathlib/Topology/List.lean,Test.lean,lake-manifest.json,lakefile.lean,lean-toolchain 7 4 ['JLimperg', 'github-actions', 'leanprover-bot'] nobody
119-23066
3 months ago
120-11386
4 months ago*
0-0
0 seconds*
21612 JLimperg
author:JLimperg
Aesop forward benchmark: master precomp Not a real PR, just for benchmarking. merge-conflict 30/27 Mathlib/Data/List/InsertIdx.lean,Mathlib/Tactic/Recall.lean,Mathlib/Topology/List.lean,Test.lean,lake-manifest.json,lakefile.lean,lean-toolchain 7 3 ['JLimperg', 'github-actions', 'leanprover-bot'] nobody
119-23065
3 months ago
120-11267
4 months ago*
0-0
0 seconds*
10678 adri326
author:adri326
feat(Topology/UniformSpace): prove that a uniform space is completely regular Provides the pseudometric definition of a uniform space (for any open set `s` and `x ∈ s`, there exists a finite family of pseudometric spaces on `X` and an `ε > 0`, such that the intersection of the balls of these pseudometric spaces is a subset of `s`), and uses it to prove that `UniformSpace X` implies `CompletelyRegularSpace X`. --- This PR aims to close the gap of pi-base's theorem [T345](https://topology.pi-base.org/theorems/T000345), which says that topological groups are completely regular. We already have a proof that topological groups are uniform, but it turns out that we do not have any connection between `UniformSpace X` and `CompletelyRegularSpace X`. There is an equivalence between `UniformSpace X` and `CompletelyRegularSpace X`: the former implies the latter, and the latter implies *the existence of* the former. This PR provides the first half of this equivalence. The construction of the pseudometric definition is based on N. Bourbaki, Chapter 9, Theorem 4.1 The proof that a uniform space is completely regular is based on [the outline on mathexchange](https://math.stackexchange.com/questions/494718/how-to-prove-that-every-uniform-space-is-completely-regular). I tried to outline the major steps of the different proofs inside of comments; I can happily be more verbose to clear up any confusion. See [the corresponding Zulip discussion](https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/Some.20missing.2C.20accessible.2C.20topology.20results) for more context. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology merge-conflict awaiting-author 332/0 Mathlib.lean,Mathlib/Topology/UniformSpace/Basic.lean,Mathlib/Topology/UniformSpace/CompletelyRegular.lean 3 6 ['ADedecker', 'adri326'] ADedecker
assignee:ADedecker
118-84993
3 months ago
118-84993
3 months ago
17-44773
17 days
20431 erdOne
author:erdOne
feat(RingTheory/AdicCompletion): monotonicity of adic-completeness --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict awaiting-author
label:t-algebra$
206/16 Mathlib.lean,Mathlib/Algebra/Module/Submodule/Defs.lean,Mathlib/Algebra/Module/Submodule/Pointwise.lean,Mathlib/RingTheory/AdicCompletion/Algebra.lean,Mathlib/RingTheory/AdicCompletion/Basic.lean,Mathlib/RingTheory/AdicCompletion/Mono.lean,Mathlib/RingTheory/Finiteness/Ideal.lean 7 13 ['chrisflav', 'erdOne', 'github-actions'] nobody
118-82478
3 months ago
118-82478
3 months ago
35-86379
35 days
18441 ADedecker
author:ADedecker
refactor(AdicTopology): use new API for algebraic filter bases, and factor some code --- - [ ] depends on: #18437 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-topology merge-conflict blocked-by-other-PR
label:t-algebra$
847/159 Mathlib.lean,Mathlib/Topology/Algebra/FilterBasis.lean,Mathlib/Topology/Algebra/FilterBasisNew.lean,Mathlib/Topology/Algebra/Nonarchimedean/AdicTopology.lean,Mathlib/Topology/Algebra/Nonarchimedean/Bases.lean,Mathlib/Topology/Algebra/Nonarchimedean/BasesNew.lean 6 3 ['ADedecker', 'github-actions', 'mathlib4-dependent-issues-bot'] nobody
117-54823
3 months ago
117-54824
3 months ago
0-679
11 minutes
20030 vihdzp
author:vihdzp
refactor: avoid ordinals in Nöbeling's theorem --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology merge-conflict WIP help-wanted 356/428 Mathlib/Topology/Category/Profinite/Nobeling.lean 1 1 ['github-actions'] nobody
117-54578
3 months ago
117-54578
3 months ago
0-0
0 seconds
18785 erdOne
author:erdOne
feat(CategoryTheory): command that generates instances for `MorphismProperty` Co-authored-by: Calle Sönne --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory t-meta merge-conflict awaiting-author 369/0 Mathlib.lean,Mathlib/CategoryTheory/MorphismProperty/Tactic.lean,MathlibTest/AddMorphismPropertyInstances.lean,scripts/noshake.json 4 19 ['alexjbest', 'chrisflav', 'erdOne', 'github-actions', 'grunweg', 'jcommelin', 'joelriou'] nobody
117-15103
3 months ago
117-15103
3 months ago
52-4682
52 days
15942 grunweg
author:grunweg
chore: move style linters into their own file; document all current linters Just to show the overall direction: this PR is just a tracking PR; it is easier to re-do the remaining pieces individually. - [x] depends on: #19529 (and needs a merge afterwards) --- The documenting of items should move into Tactic.Linter... [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-linter merge-conflict awaiting-author 634/287 Mathlib.lean,Mathlib/Analysis/SpecialFunctions/BinaryEntropy.lean,Mathlib/Geometry/Manifold/Instances/Real.lean,Mathlib/Init.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Common.lean,Mathlib/Tactic/Linter.lean,Mathlib/Tactic/Linter/AdmitLinter.lean,Mathlib/Tactic/Linter/GlobalAttributeIn.lean,Mathlib/Tactic/Linter/HashCommandLinter.lean,Mathlib/Tactic/Linter/HaveLetLinter.lean,Mathlib/Tactic/Linter/Lint.lean,Mathlib/Tactic/Linter/OldObtain.lean,Mathlib/Tactic/Linter/RefineLinter.lean,Mathlib/Tactic/Linter/Style.lean,Mathlib/Tactic/Linter/UnusedTactic.lean,Mathlib/Util/SleepHeartbeats.lean,lakefile.lean,test/AdmitLinter.lean,test/Change.lean,test/Check.lean,test/Clear!.lean,test/ClearExcept.lean,test/Clear_.lean,test/DefEqTransformations.lean,test/DeriveToExpr.lean,test/ExtractGoal.lean,test/ExtractLets.lean,test/GuardGoalNums.lean,test/GuardHypNums.lean,test/HashCommandLinter.lean,test/Lint.lean,test/LintStyle.lean,test/MfldSetTac.lean,test/MinImports.lean,test/SimpRw.lean,test/SplitIfs.lean,test/TermBeta.lean,test/TypeCheck.lean,test/UnsetOption.lean,test/Use.lean,test/basicTactics.lean,test/casesm.lean,test/convert.lean,test/fail_if_no_progress.lean,test/fun_prop_dev.lean,test/itauto.lean,test/meta.lean,test/notation3.lean,test/recover.lean,test/says.lean,test/symm.lean,test/trace.lean,test/trans.lean 54 5 ['github-actions', 'grunweg', 'joneugster', 'mathlib4-dependent-issues-bot'] nobody
115-41727
3 months ago
115-41727
3 months ago
0-36287
10 hours
21746 robin-carlier
author:robin-carlier
feat(AlgebraicTopology/SimplexCategory/GeneratorsRelations/NormalForms): Normal forms for `P_δ`s We prove that admissible lists indeed provide a normal form for morphisms of satisfying `P_δ`. To this end, we introduce `standardδ`, a construction that takes a list and turn it into a composition of `δ i`s in `SimplexCategoryGenRel`. We then prove that, thanks to the first simplicial identity, composition on the left corresponds to simplicial insertion in the list. This gives existence of a normal form for every morphism satisfying `P_δ`. For unicity, we introduce an auxiliary function `simplicialEvalδ : (List ℕ) → ℕ → ℕ` and show that for admissible lists, it lifts to `ℕ` the `orderHom` attached to `toSimplexCategory.map standardδ`, and that we can recover elements of the list only by looking at values of this function. Part of a series of PR formalising that `SimplexCategoryGenRel` is equivalent to `SimplexCategory`. --- - [ ] depends on: #21745 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology t-category-theory merge-conflict blocked-by-other-PR 1458/0 Mathlib.lean,Mathlib/AlgebraicTopology/SimplexCategory/GeneratorsRelations/Basic.lean,Mathlib/AlgebraicTopology/SimplexCategory/GeneratorsRelations/EpiMono.lean,Mathlib/AlgebraicTopology/SimplexCategory/GeneratorsRelations/NormalForms.lean 4 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
115-39352
3 months ago
115-39352
3 months ago
0-1140
19 minutes
21747 robin-carlier
author:robin-carlier
feat(AlgebraicTopology/SimplexCategory/GeneratorsRelations): `SimplexCategoryGenRel.toSimplexCategory` is an equivalence We use the normal forms for morphisms in `SimplexCategoryGenRel` to prove that `SimplexCategoryGenRel.toSimplexCategory` is an equivalence. We prove in order that there exists unique lifts in `SimplexCategoryGenRel` of mono (resp. epis) in `SimplexCategory`, and use this to deduce fully faithfulness of `SimplexCategoryGenRel.toSimplexCategory` thanks to the existing epi-mono factorisation in `SimplexCategory`. Part of a series of PR formalising that `SimplexCategoryGenRel` is equivalent to `SimplexCategory`. --- - [ ] depends on: #21746 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology t-category-theory merge-conflict blocked-by-other-PR 1832/0 Mathlib.lean,Mathlib/AlgebraicTopology/SimplexCategory/GeneratorsRelations/Basic.lean,Mathlib/AlgebraicTopology/SimplexCategory/GeneratorsRelations/EpiMono.lean,Mathlib/AlgebraicTopology/SimplexCategory/GeneratorsRelations/Equivalence.lean,Mathlib/AlgebraicTopology/SimplexCategory/GeneratorsRelations/NormalForms.lean 5 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
115-39351
3 months ago
115-39351
3 months ago
0-1054
17 minutes
21748 robin-carlier
author:robin-carlier
feat(AlgebraicTopology/SimplexCategory/SimplicialObject): definitions of simplicial objects by generators and relation We leverage the equivalence between `SimplexCategory` and `SimplexCategoryGenRel` to give new constructors for (co)simplicial objects, as well as constructors for natural transformations (resp. isomorphism) between those. Final PR in the series of PR formalising the equivalence between `SimplexCategory` and `SimplexCategoryGenRel`. --- - [ ] depends on: #21747 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology t-category-theory merge-conflict blocked-by-other-PR 2253/0 Mathlib.lean,Mathlib/AlgebraicTopology/SimplexCategory/GeneratorsRelations/Basic.lean,Mathlib/AlgebraicTopology/SimplexCategory/GeneratorsRelations/EpiMono.lean,Mathlib/AlgebraicTopology/SimplexCategory/GeneratorsRelations/Equivalence.lean,Mathlib/AlgebraicTopology/SimplexCategory/GeneratorsRelations/NormalForms.lean,Mathlib/AlgebraicTopology/SimplicialObject/GeneratorsRelations.lean 6 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
115-39350
3 months ago
115-39350
3 months ago
0-976
16 minutes
20334 miguelmarco
author:miguelmarco
feat: allow polyrith to use a local Singular/Sage install Try to call a local install of Singular (either standalone or inside Sage) to find the witness for polyrith before trying to call the online sage cell server. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-meta merge-conflict awaiting-author 171/48 Mathlib/Tactic/Polyrith.lean,scripts/polyrith_sage.py 2 13 ['eric-wieser', 'github-actions', 'hanwenzhu', 'kim-em', 'miguelmarco'] nobody
115-38253
3 months ago
115-38253
3 months ago
27-65384
27 days
16311 madvorak
author:madvorak
feat(Computability): regular languages are context-free --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-computability merge-conflict WIP 72/0 Mathlib.lean,Mathlib/Computability/Chomsky.lean,Mathlib/Computability/ContextFreeGrammar.lean 3 7 ['Rida-Hamadani', 'YaelDillies', 'github-actions', 'madvorak'] nobody
115-21522
3 months ago
115-21522
3 months ago
0-0
0 seconds
19943 AlexLoitzl
author:AlexLoitzl
feat(Computability): Add Chomsky Normal Form Grammar and translation - Define Chomsky normal form grammars - Add language-preserving translation between context-free grammars and Chomsky normal form grammars Co-authored-by: Martin Dvorak martin.dvorak@matfyz.cz --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-computability new-contributor merge-conflict awaiting-author 3151/0 Mathlib.lean,Mathlib/Computability/ChomskyNormalForm/Basic.lean,Mathlib/Computability/ChomskyNormalForm/EmptyElimination.lean,Mathlib/Computability/ChomskyNormalForm/LengthRestriction.lean,Mathlib/Computability/ChomskyNormalForm/TerminalRestriction.lean,Mathlib/Computability/ChomskyNormalForm/Translation.lean,Mathlib/Computability/ChomskyNormalForm/UnitElimination.lean,Mathlib/Computability/ContextFreeGrammar.lean 8 59 ['AlexLoitzl', 'YaelDillies', 'github-actions', 'kim-em', 'madvorak'] nobody
115-21275
3 months ago
115-21275
3 months ago
37-29014
37 days
19616 adamtopaz
author:adamtopaz
fix: Fix the definition of the absolute Galois group of a field Previously it was defined as the Galois group of the algebraic closure, as opposed to the separable closure. Also, this adds some missing instances for this group. Still missing is compactness, but that seems like a bigger project. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-number-theory merge-conflict awaiting-author
label:t-algebra$
23/8 Mathlib/FieldTheory/AbsoluteGaloisGroup.lean,Mathlib/FieldTheory/KrullTopology.lean 2 4 ['acmepjz', 'alreadydone', 'github-actions'] nobody
115-19510
3 months ago
115-19510
3 months ago
3-64280
3 days
19802 vihdzp
author:vihdzp
refactor(SetTheory/Ordinal/Arithmetic): `Ordinal.IsLimit` → `Order.IsSuccLimit` This is part of a series of ordinal refactors which aim to replace definitions specific to `Ordinal` with more general concepts. See #17033 for more info. --- - [x] depends on: #19800 - [x] depends on: #19801 - [x] depends on: #19916 - [ ] depends on: #21751 Took us long enough. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-set-theory t-order merge-conflict awaiting-author blocked-by-other-PR 513/335 Mathlib/MeasureTheory/MeasurableSpace/Card.lean,Mathlib/Order/SuccPred/Limit.lean,Mathlib/SetTheory/Cardinal/Aleph.lean,Mathlib/SetTheory/Cardinal/Arithmetic.lean,Mathlib/SetTheory/Cardinal/Cofinality.lean,Mathlib/SetTheory/Game/Birthday.lean,Mathlib/SetTheory/Ordinal/Arithmetic.lean,Mathlib/SetTheory/Ordinal/Exponential.lean,Mathlib/SetTheory/Ordinal/FixedPoint.lean,Mathlib/SetTheory/Ordinal/Notation.lean,Mathlib/SetTheory/Ordinal/Principal.lean,Mathlib/SetTheory/Ordinal/Topology.lean,Mathlib/Topology/Category/Profinite/Nobeling.lean 13 10 ['YaelDillies', 'github-actions', 'kim-em', 'mathlib4-dependent-issues-bot', 'vihdzp'] nobody
114-12189
3 months ago
114-12189
3 months ago
33-82297
33 days
18439 ADedecker
author:ADedecker
refactor: use new algebraic filter bases API in `FiniteAdeleRing` --- - [ ] depends on: #18437 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-topology merge-conflict blocked-by-other-PR
label:t-algebra$
699/21 Mathlib.lean,Mathlib/RingTheory/DedekindDomain/FiniteAdeleRing.lean,Mathlib/Topology/Algebra/FilterBasis.lean,Mathlib/Topology/Algebra/FilterBasisNew.lean,Mathlib/Topology/Algebra/Nonarchimedean/Bases.lean,Mathlib/Topology/Algebra/Nonarchimedean/BasesNew.lean 6 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
113-12352
3 months ago
113-12352
3 months ago
0-619
10 minutes
21761 JovanGerb
author:JovanGerb
feat(Algebra): add lemmas `mul_self` and `add_self` This is point (4) in https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Possible.20improvements.20to.20Lean.2FMathlib/near/499085779 I decided to go with `n + n = 2 * n` instead of `n + n = n * 2` because it feels more natural. Feel free to suggest the opposite. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict delegated
label:t-algebra$
206/196 Archive/Imo/Imo1959Q2.lean,Archive/Imo/Imo1961Q3.lean,Archive/Imo/Imo2008Q4.lean,Archive/Imo/Imo2013Q1.lean,Archive/Imo/Imo2024Q3.lean,Archive/MiuLanguage/DecisionSuf.lean,Archive/Wiedijk100Theorems/Partition.lean,Archive/ZagierTwoSquares.lean,Mathlib/Algebra/CharP/Two.lean,Mathlib/Algebra/CharZero/Lemmas.lean,Mathlib/Algebra/Group/Defs.lean,Mathlib/Algebra/Group/Even.lean,Mathlib/Algebra/Lie/Weights/RootSystem.lean,Mathlib/Algebra/Order/Field/Basic.lean,Mathlib/Algebra/Order/Group/Lattice.lean,Mathlib/Algebra/Order/Group/Unbundled/Abs.lean,Mathlib/Algebra/Order/Ring/Basic.lean,Mathlib/Algebra/Order/Ring/Unbundled/Basic.lean,Mathlib/Algebra/Order/Round.lean,Mathlib/Algebra/Polynomial/Taylor.lean,Mathlib/Algebra/Ring/BooleanRing.lean,Mathlib/Algebra/Ring/Defs.lean,Mathlib/Algebra/Ring/Hom/Defs.lean,Mathlib/Algebra/Ring/Int/Parity.lean,Mathlib/Algebra/Ring/Invertible.lean,Mathlib/Algebra/Ring/Parity.lean,Mathlib/Algebra/Ring/SumsOfSquares.lean,Mathlib/Algebra/Symmetrized.lean,Mathlib/Algebra/Tropical/Basic.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Jacobian.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Projective.lean,Mathlib/Analysis/CStarAlgebra/CStarMatrix.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Order.lean,Mathlib/Analysis/Complex/Isometry.lean,Mathlib/Analysis/Complex/PhragmenLindelof.lean,Mathlib/Analysis/Complex/UpperHalfPlane/Metric.lean,Mathlib/Analysis/Convex/Mul.lean,Mathlib/Analysis/Convex/SpecificFunctions/Deriv.lean,Mathlib/Analysis/InnerProductSpace/LinearMap.lean,Mathlib/Analysis/Normed/Lp/ProdLp.lean,Mathlib/Analysis/NormedSpace/MStructure.lean,Mathlib/Analysis/RCLike/Basic.lean,Mathlib/Analysis/SpecialFunctions/Bernstein.lean,Mathlib/Analysis/SpecialFunctions/BinaryEntropy.lean,Mathlib/Analysis/SpecialFunctions/Complex/Arctan.lean,Mathlib/Analysis/SpecialFunctions/Complex/Arg.lean,Mathlib/Analysis/SpecialFunctions/Gamma/Beta.lean,Mathlib/Analysis/SpecialFunctions/Gaussian/GaussianIntegral.lean,Mathlib/Analysis/SpecialFunctions/PolarCoord.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Angle.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Series.lean,Mathlib/Combinatorics/Additive/AP/Three/Defs.lean,Mathlib/Combinatorics/SetFamily/HarrisKleitman.lean,Mathlib/Combinatorics/SimpleGraph/DegreeSum.lean,Mathlib/Combinatorics/SimpleGraph/Matching.lean,Mathlib/Computability/AkraBazzi/AkraBazzi.lean,Mathlib/Computability/Language.lean,Mathlib/Data/Complex/Abs.lean,Mathlib/Data/Complex/Module.lean,Mathlib/Data/Complex/Norm.lean,Mathlib/Data/ENNReal/Holder.lean,Mathlib/Data/ENNReal/Inv.lean,Mathlib/Data/Nat/Bitwise.lean,Mathlib/Data/Nat/Cast/Order/Ring.lean,Mathlib/Data/Nat/Choose/Central.lean,Mathlib/Data/Num/Lemmas.lean,Mathlib/Data/Num/Prime.lean,Mathlib/Data/Real/Pi/Irrational.lean,Mathlib/Data/ZMod/Basic.lean,Mathlib/Dynamics/Circle/RotationNumber/TranslationNumber.lean,Mathlib/FieldTheory/Finite/Basic.lean,Mathlib/Geometry/Euclidean/Angle/Oriented/RightAngle.lean,Mathlib/Geometry/Euclidean/Angle/Unoriented/RightAngle.lean,Mathlib/GroupTheory/Coxeter/Inversion.lean,Mathlib/GroupTheory/Perm/Cycle/Type.lean,Mathlib/GroupTheory/SpecificGroups/Alternating.lean,Mathlib/GroupTheory/SpecificGroups/Dihedral.lean,Mathlib/GroupTheory/SpecificGroups/KleinFour.lean,Mathlib/LinearAlgebra/AffineSpace/Midpoint.lean,Mathlib/LinearAlgebra/Matrix/Charpoly/Eigs.lean,Mathlib/LinearAlgebra/Matrix/PosDef.lean,Mathlib/LinearAlgebra/QuadraticForm/Complex.lean,Mathlib/LinearAlgebra/SesquilinearForm.lean,Mathlib/MeasureTheory/Function/L1Space/HasFiniteIntegral.lean,Mathlib/MeasureTheory/Integral/Bochner.lean,Mathlib/MeasureTheory/Integral/Gamma.lean,Mathlib/MeasureTheory/Measure/LevyProkhorovMetric.lean,Mathlib/NumberTheory/Cyclotomic/Embeddings.lean,Mathlib/NumberTheory/FLT/Three.lean,Mathlib/NumberTheory/GaussSum.lean,Mathlib/NumberTheory/LegendreSymbol/Basic.lean,Mathlib/NumberTheory/LegendreSymbol/JacobiSymbol.lean,Mathlib/NumberTheory/LegendreSymbol/QuadraticChar/Basic.lean,Mathlib/NumberTheory/LegendreSymbol/QuadraticReciprocity.lean,Mathlib/NumberTheory/ModularForms/EisensteinSeries/UniformConvergence.lean,Mathlib/NumberTheory/Multiplicity.lean,Mathlib/NumberTheory/NumberField/Basic.lean,Mathlib/NumberTheory/NumberField/CanonicalEmbedding/ConvexBody.lean,Mathlib/NumberTheory/PellMatiyasevic.lean,Mathlib/NumberTheory/SumPrimeReciprocals.lean 117 13 ['JovanGerb', 'YaelDillies', 'github-actions', 'grunweg', 'mathlib-bors', 'riccardobrasca'] nobody
112-82253
3 months ago
113-27024
3 months ago
0-54729
15 hours
17005 YnirPaz
author:YnirPaz
feat(SetTheory/Cardinal/Regular): define singular cardinals Define singular cardinals and prove basic lemmas about them. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-set-theory merge-conflict WIP 94/1 Mathlib.lean,Mathlib/SetTheory/Cardinal/Regular.lean,Mathlib/SetTheory/Ordinal/Basic.lean 3 28 ['YaelDillies', 'YnirPaz', 'github-actions', 'vihdzp'] nobody
112-54631
3 months ago
188-47813
6 months ago
34-18388
34 days
20180 ChrisHughes24
author:ChrisHughes24
feat(ModelTheory): definable functions --- Possibly this should be generalized to partial functions. - [x] depends on: #20166 - [ ] depends on: #20161 - [x] depends on: #20115 - [x] depends on: #20174 - [ ] depends on: #20175 - [ ] depends on: #21948 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-logic merge-conflict blocked-by-other-PR 671/1 Mathlib.lean,Mathlib/ModelTheory/FunctionalFormula.lean,Mathlib/ModelTheory/Semantics.lean,Mathlib/ModelTheory/Syntax.lean 4 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
112-19817
3 months ago
112-19817
3 months ago
0-563
9 minutes
20173 ChrisHughes24
author:ChrisHughes24
refactor(ModelTheory): tidy up proof of Ax-Grothendieck with definable functions --- - [x] depends on: #20166 - [x] depends on: #20161 - [x] depends on: #20115 - [x] depends on: #20174 - [ ] depends on: #20175 - [ ] depends on: #20180 - [ ] depends on: #21948 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-logic merge-conflict blocked-by-other-PR 671/1 Mathlib.lean,Mathlib/ModelTheory/FunctionalFormula.lean,Mathlib/ModelTheory/Semantics.lean,Mathlib/ModelTheory/Syntax.lean 4 6 ['ChrisHughes24', 'github-actions', 'mathlib4-dependent-issues-bot'] nobody
112-19817
3 months ago
112-19817
3 months ago
0-0
0 seconds
21948 ChrisHughes24
author:ChrisHughes24
feat(ModelTheory): Formula.iSup and iInf --- This was a slightly controversial addition discussed in #20175 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-logic merge-conflict 24/7 Mathlib/ModelTheory/Semantics.lean,Mathlib/ModelTheory/Syntax.lean 2 5 ['YaelDillies', 'github-actions'] nobody
112-19326
3 months ago
112-19326
3 months ago
1-18127
1 day
18952 Command-Master
author:Command-Master
chore: deprecate `Trunc` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data merge-conflict WIP 283/57 Mathlib/CategoryTheory/EpiMono.lean,Mathlib/CategoryTheory/Preadditive/Biproducts.lean,Mathlib/Data/DFinsupp/Defs.lean,Mathlib/Data/Fintype/Basic.lean,Mathlib/Data/Fintype/Option.lean,Mathlib/Data/Fintype/Quotient.lean,Mathlib/Data/Quot.lean,Mathlib/Data/Semiquot.lean,Mathlib/GroupTheory/Perm/Cycle/Factors.lean,Mathlib/GroupTheory/Perm/Sign.lean,Mathlib/LinearAlgebra/Determinant.lean,Mathlib/Logic/Equiv/List.lean 12 8 ['eric-wieser', 'github-actions', 'vihdzp'] nobody
112-5848
3 months ago
112-5848
3 months ago
0-0
0 seconds
18206 vihdzp
author:vihdzp
chore(SetTheory/Ordinal/Basic): golf/clean up `Cardinal.ord` theorems --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-set-theory merge-conflict awaiting-author 48/57 Mathlib/SetTheory/Ordinal/Basic.lean 1 5 ['alreadydone', 'github-actions', 'urkud', 'vihdzp'] nobody
110-54009
3 months ago
110-54009
3 months ago
81-35878
81 days
18463 vihdzp
author:vihdzp
feat(SetTheory/Ordinal/Notation/FundamentalSequence): define type of fundamental sequences We define `Sequence α` as the type of sequences with length 0, 1, or `ω`, and give a basic API. A subsequent PR will introduce the notion of a (countable and computable) fundamental sequence and establish basic results. The goal of this is to generalize [`ONote.fundamentalSequence`](https://leanprover-community.github.io/mathlib4_docs/Mathlib/SetTheory/Ordinal/Notation.html#ONote.fundamentalSequence) to allow the construction of fundamental sequences for other ordinal notations. --- See [my ordinal notation repository](https://github.com/vihdzp/ordinal-notation/blob/a6fdd7fe7cb521e686ea271902e7e5496f1804d3/OrdinalNotation/Cantor.lean#L1218) for a demonstration of how this API looks in practice. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-set-theory t-order merge-conflict 174/1 Mathlib.lean,Mathlib/SetTheory/Ordinal/Notation/Cantor.lean,Mathlib/SetTheory/Ordinal/Notation/FundamentalSequence.lean 3 19 ['YnirPaz', 'b-mehta', 'github-actions', 'vihdzp'] nobody
110-54008
3 months ago
110-54008
3 months ago
52-25108
52 days
10541 Louddy
author:Louddy
feat(Algebra/SkewMonoidAlgebra/Basic): add SkewMonoidAlgebra # Skew Monoid algebras This file presents a skewed version of `Mathlib.Algebra.MonoidAlgebra.Basic`. ## Definition We define `SkewMonoidAlgebra k G := G →₀ k` attached with a skewed convolution product. Here, the product of two elements `f g : SkewMonoidAlgebra k G` is the finitely supported function whose value at `a` is the sum of `f x * (x • g y)` over all pairs `x, y` such that `x * y = a`. This will be used in a later PR to define skew polynomial rings. Co-authored-by: María Inés de Frutos Fernández <[mariaines.dff@gmail.com](mailto:mariaines.dff@gmail.com)> --- - [x] depends on: #15878 - [x] depends on: #19084 - [ ] depends on: #22078 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra merge-conflict blocked-by-other-PR WIP
label:t-algebra$
1624/0 Mathlib.lean,Mathlib/Algebra/Group/InjSurj.lean,Mathlib/Algebra/SkewMonoidAlgebra/Basic.lean,Mathlib/Algebra/SkewMonoidAlgebra/Lift.lean 4 105 ['AntoineChambert-Loir', 'Louddy', 'YaelDillies', 'eric-wieser', 'fpvandoorn', 'github-actions', 'mariainesdff', 'mathlib4-dependent-issues-bot', 'mattrobball'] AntoineChambert-Loir
assignee:AntoineChambert-Loir
110-24901
3 months ago
110-24902
3 months ago
179-12934
179 days
12054 adomani
author:adomani
feat: auto-bugs This PR introduces a linter for suggesting bugs in tactics. See * #12077 * #12083 * #12084 for some bugs exposed by the test suite. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta merge-conflict awaiting-author 737/0 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter/MetaTesting.lean,scripts/noshake.json,test/MetaTesting.lean 5 20 ['adomani', 'eric-wieser', 'github-actions', 'joneugster', 'kim-em'] joneugster
assignee:joneugster
109-64103
3 months ago
109-64103
3 months ago
45-6057
45 days
5062 adomani
author:adomani
feat(Tactic/Prune + test/Prune): add `prune` tactic, for removing unnecessary hypotheses This tactic removes very conservatively all local declarations that 1. do not appear in the main goal, 2. do not appear in a declaration that appears in the main goal, 3. ... and so on recursively. The main motivation for this tactic is that all available variables in the current `namespace/section` appear in the goal state, not just the ones that are needed for the statement to type-check. Using `prune` mitigates this situation. The tactic also admits an optional natural number argument: `prune n` removes all variables that have not appeared at the `(n+1)`-st stage in the above list. Thus, `prune 0` only leaves the variables needed for the statement to type-check. Also, for sufficiently large `n`, `prune n` is a synonym for `prune`. [Zulip discussion](https://leanprover.zulipchat.com/#narrow/stream/270676-lean4/topic/substitute.20for.20.60include.2Fomit.60.3F) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta merge-conflict modifies-tactic-syntax awaiting-author 181/0 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Prune.lean,test/Prune.lean 4 5 ['adomani', 'j-loreaux', 'kmill'] nobody
109-31410
3 months ago
109-31410
3 months ago
195-56460
195 days
21914 vasnesterov
author:vasnesterov
Test PR for `order` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import merge-conflict WIP 2052/1507 Mathlib.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/ExtClass.lean,Mathlib/Algebra/Homology/Embedding/CochainComplex.lean,Mathlib/Algebra/Homology/ExactSequence.lean,Mathlib/Algebra/Homology/HomotopyCategory/DegreewiseSplit.lean,Mathlib/Algebra/Homology/HomotopyCategory/HomComplex.lean,Mathlib/Algebra/Homology/HomotopyCategory/HomComplexShift.lean,Mathlib/Algebra/Homology/HomotopyCategory/MappingCone.lean,Mathlib/Algebra/Homology/HomotopyCategory/Pretriangulated.lean,Mathlib/Algebra/Homology/HomotopyCategory/Triangulated.lean,Mathlib/AlgebraicTopology/SimplexCategory/Basic.lean,Mathlib/AlgebraicTopology/SimplexCategory/MorphismProperty.lean,Mathlib/AlgebraicTopology/SimplicialSet/Coskeletal.lean,Mathlib/AlgebraicTopology/SimplicialSet/Path.lean,Mathlib/Analysis/Convex/Radon.lean,Mathlib/Analysis/Convex/Slope.lean,Mathlib/Analysis/Normed/Affine/Simplex.lean,Mathlib/Analysis/SpecialFunctions/BinaryEntropy.lean,Mathlib/Analysis/SpecialFunctions/Log/Base.lean,Mathlib/Analysis/SpecialFunctions/Log/Monotone.lean,Mathlib/CategoryTheory/Abelian/ProjectiveDimension.lean,Mathlib/CategoryTheory/Functor/OfSequence.lean,Mathlib/CategoryTheory/Limits/Shapes/SequentialProduct.lean,Mathlib/Combinatorics/Schnirelmann.lean,Mathlib/Combinatorics/SetFamily/KruskalKatona.lean,Mathlib/Combinatorics/SimpleGraph/Connectivity/Subgraph.lean,Mathlib/Computability/AkraBazzi/GrowsPolynomially.lean,Mathlib/Data/Finset/Card.lean,Mathlib/Data/List/Nodup.lean,Mathlib/Data/Rat/Lemmas.lean,Mathlib/GroupTheory/Coxeter/Basic.lean,Mathlib/GroupTheory/Coxeter/Inversion.lean,Mathlib/GroupTheory/Coxeter/Length.lean,Mathlib/GroupTheory/Exponent.lean,Mathlib/MeasureTheory/Integral/PeakFunction.lean,Mathlib/MeasureTheory/Measure/Lebesgue/VolumeOfBalls.lean,Mathlib/MeasureTheory/Measure/LevyProkhorovMetric.lean,Mathlib/NumberTheory/ClassNumber/Finite.lean,Mathlib/NumberTheory/Fermat.lean,Mathlib/NumberTheory/FermatPsp.lean,Mathlib/NumberTheory/Modular.lean,Mathlib/NumberTheory/NumberField/Embeddings.lean,Mathlib/NumberTheory/NumberField/FinitePlaces.lean,Mathlib/NumberTheory/Padics/PadicVal/Basic.lean,Mathlib/Order/Basic.lean,Mathlib/Order/BasicLemmas.lean,Mathlib/Order/KrullDimension.lean,Mathlib/Order/RelSeries.lean,Mathlib/Probability/Distributions/Exponential.lean,Mathlib/Probability/Distributions/Gamma.lean,Mathlib/Probability/Distributions/Pareto.lean,Mathlib/Probability/StrongLaw.lean,Mathlib/RingTheory/AdicCompletion/Exactness.lean,Mathlib/RingTheory/Filtration.lean,Mathlib/RingTheory/PowerSeries/Basic.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Order.lean,MathlibTest/order.lean 58 4 ['github-actions', 'leanprover-bot', 'vasnesterov'] nobody
109-13157
3 months ago
109-13158
3 months ago
0-0
0 seconds
16705 iehality
author:iehality
feat(Computability): r.e. sets are closed under inter/union/projection/composition Prove that r.e. sets are closed under intersections, unions, projection and composition. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-computability merge-conflict awaiting-author 130/0 Mathlib/Computability/Halting.lean 1 3 ['YaelDillies', 'github-actions'] nobody
108-17910
3 months ago
108-17910
3 months ago
68-14150
68 days
22169 JLimperg
author:JLimperg
Aesop forward benchmark: forward no-precomp naive Not a real PR, just for benchmarking. merge-conflict 31/27 Mathlib/Data/List/InsertIdx.lean,Mathlib/Tactic/Recall.lean,Mathlib/Topology/List.lean,Test.lean,lake-manifest.json,lakefile.lean,lean-toolchain 7 6 ['JLimperg', 'github-actions', 'leanprover-bot'] nobody
107-83474
3 months ago
108-9128
3 months ago*
0-0
0 seconds*
21433 grunweg
author:grunweg
chore: change more lemmas to be about enorm instead of nnnorm --- - [x] depends on: #21782 - [x] depends on: #21783 (and this PR modifies the file split, and file splits are painful to merge over) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) carleson t-measure-probability merge-conflict awaiting-author 172/71 Mathlib/Analysis/Distribution/SchwartzSpace.lean,Mathlib/Analysis/Normed/Group/Basic.lean,Mathlib/Analysis/SpecialFunctions/Pow/NNReal.lean,Mathlib/Data/ENNReal/Basic.lean,Mathlib/MeasureTheory/Function/LpSeminorm/Basic.lean,Mathlib/MeasureTheory/Function/LpSeminorm/CompareExp.lean,Mathlib/MeasureTheory/Function/LpSpace/Basic.lean,Mathlib/MeasureTheory/Function/LpSpace/ContinuousFunctions.lean,Mathlib/MeasureTheory/Function/UniformIntegrable.lean 9 18 ['RemyDegenne', 'github-actions', 'grunweg', 'j-loreaux', 'mathlib4-dependent-issues-bot'] nobody
107-82663
3 months ago
110-29747
3 months ago
2-42743
2 days
22171 JLimperg
author:JLimperg
Aesop forward benchmark: forward no-precomp naive rpinf pr-release Not a real PR, just for benchmarking. merge-conflict 31/27 Mathlib/Data/List/InsertIdx.lean,Mathlib/Tactic/Recall.lean,Mathlib/Topology/List.lean,Test.lean,lake-manifest.json,lakefile.lean,lean-toolchain 7 5 ['JLimperg', 'github-actions', 'leanprover-bot'] nobody
107-4947
3 months ago
108-8691
3 months ago*
0-0
0 seconds*
21099 chrisflav
author:chrisflav
chore(RingTheory/Generators): use unification hints for variables and relations When working with generators and presentations, we rely on the `MvPolynomial` API, but since the type of variables is bundled in `Generators R S`, many lemmas don't apply with `rw` or `simp`, because they can't see through the definition of `vars` in constructions such as `Generators.comp` and `Generators.localizationAway`. A possible approach is to make all of these constructions `abbrev`s, but this causes `simp` to also unfold `val` which is not always desirable. More generally, it is then harder to predict how instance search and `simp` behave. This approach is tried in #21050, but causes many regressions. This approach is less invasive, as it uses `unif_hint` to unify the `vars` (and `rels`) fields of constructions with the correct type. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict
label:t-algebra$
231/91 Mathlib/Algebra/Module/Presentation/Differentials.lean,Mathlib/RingTheory/Generators.lean,Mathlib/RingTheory/Kaehler/JacobiZariski.lean,Mathlib/RingTheory/Presentation.lean,Mathlib/RingTheory/Smooth/StandardSmooth.lean 5 16 ['chrisflav', 'erdOne', 'github-actions', 'leanprover-bot', 'mattrobball'] nobody
106-12844
3 months ago
106-12844
3 months ago
27-75210
27 days
21269 CharredLee
author:CharredLee
(WIP) feat (CategoryTheory/Topos): Add topos theory content This code contains basic definitions and results in topos theory, including the definition of a subobject classifier, power objects, and topoi. It is proved that every topos has exponential objects, i.e. "internal homs". The mathematical content follows chapter IV sections 1-2 of Mac Lane and Moerdijk's text "Sheaves in Geometry and Logic". --- - [x] depends on: #21281 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-category-theory merge-conflict awaiting-author WIP 1269/0 Mathlib.lean,Mathlib/CategoryTheory/Topos/Basic.lean,Mathlib/CategoryTheory/Topos/Classifier.lean,Mathlib/CategoryTheory/Topos/Exponentials.lean,Mathlib/CategoryTheory/Topos/Power.lean 5 10 ['CharredLee', 'gio256', 'github-actions', 'joelriou', 'mathlib4-dependent-issues-bot'] nobody
104-73947
3 months ago
104-73947
3 months ago
0-13879
3 hours
12394 JADekker
author:JADekker
feat : define pre-tight and tight measures Define tight measures (by first defining separable and pre-tight measures). Define some api for all three concepts Prove Ulam's tightness theorem and a strengthened version of this. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-measure-probability merge-conflict please-adopt awaiting-author 503/0 Mathlib.lean,Mathlib/MeasureTheory/Measure/Tight.lean 2 34 ['EtienneC30', 'JADekker', 'github-actions', 'sgouezel'] nobody
104-16440
3 months ago
104-16440
3 months ago
2-604
2 days
22245 Champitoad
author:Champitoad
feat(CategoryTheory/Subobject): add formalization of subobject classifier This introduces a file `Classifier.lean` defining the notion `Classifier C` of subobject classifier in any category `C` with a terminal object, following Section I.3 of "Sheaves in Geometry and Logic" [MM92]. This is related to but independent from #21281, because our definition associates a characteristic map to every _subobject_ rather than every _monomorphism_. Adopting this "extensional" rather than "intensional" definition allows us to formalize the proof of Proposition 1 in [MM92, Section I.3] (`hasClassifier_isRepresentable_iff`), that `C` has a subobject classifier if and only if the subobjects presheaf `sub C` is representable. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-category-theory merge-conflict awaiting-author 5219/2536 Cache/Hashing.lean,Cache/IO.lean,Cache/Lean.lean,Mathlib.lean,Mathlib/Algebra/Algebra/Defs.lean,Mathlib/Algebra/Category/AlgebraCat/Limits.lean,Mathlib/Algebra/Category/BoolRing.lean,Mathlib/Algebra/Category/FGModuleCat/Basic.lean,Mathlib/Algebra/Category/Grp/AB.lean,Mathlib/Algebra/Category/Grp/EpiMono.lean,Mathlib/Algebra/Category/HopfAlgebraCat/Monoidal.lean,Mathlib/Algebra/Category/ModuleCat/Abelian.lean,Mathlib/Algebra/Category/ModuleCat/Adjunctions.lean,Mathlib/Algebra/Category/ModuleCat/Basic.lean,Mathlib/Algebra/Category/ModuleCat/Biproducts.lean,Mathlib/Algebra/Category/ModuleCat/ChangeOfRings.lean,Mathlib/Algebra/Category/ModuleCat/Differentials/Basic.lean,Mathlib/Algebra/Category/ModuleCat/EpiMono.lean,Mathlib/Algebra/Category/ModuleCat/FilteredColimits.lean,Mathlib/Algebra/Category/ModuleCat/Kernels.lean,Mathlib/Algebra/Category/ModuleCat/Monoidal/Basic.lean,Mathlib/Algebra/Category/ModuleCat/Presheaf/Colimits.lean,Mathlib/Algebra/Category/ModuleCat/Presheaf/Limits.lean,Mathlib/Algebra/Category/ModuleCat/Subobject.lean,Mathlib/Algebra/Category/MonCat/FilteredColimits.lean,Mathlib/Algebra/Category/Ring/Colimits.lean,Mathlib/Algebra/Category/Ring/Limits.lean,Mathlib/Algebra/Group/Commute/Units.lean,Mathlib/Algebra/Group/Pointwise/Set/Card.lean,Mathlib/Algebra/Homology/ComplexShape.lean,Mathlib/Algebra/Homology/Double.lean,Mathlib/Algebra/Homology/HasNoLoop.lean,Mathlib/Algebra/Homology/Homotopy.lean,Mathlib/Algebra/Polynomial/Basic.lean,Mathlib/Algebra/Polynomial/Degree/Operations.lean,Mathlib/Algebra/Polynomial/Lifts.lean,Mathlib/Algebra/Polynomial/Sequence.lean,Mathlib/AlgebraicTopology/SimplexCategory/GeneratorsRelations/EpiMono.lean,Mathlib/Analysis/CStarAlgebra/Spectrum.lean,Mathlib/Analysis/Complex/AbelLimit.lean,Mathlib/Analysis/Complex/AbsMax.lean,Mathlib/Analysis/Complex/Angle.lean,Mathlib/Analysis/Complex/Arg.lean,Mathlib/Analysis/Complex/Basic.lean,Mathlib/Analysis/Complex/CauchyIntegral.lean,Mathlib/Analysis/Complex/Circle.lean,Mathlib/Analysis/Complex/Hadamard.lean,Mathlib/Analysis/Complex/Isometry.lean,Mathlib/Analysis/Complex/Liouville.lean,Mathlib/Analysis/Complex/LocallyUniformLimit.lean,Mathlib/Analysis/Complex/OpenMapping.lean,Mathlib/Analysis/Complex/Periodic.lean,Mathlib/Analysis/Complex/PhragmenLindelof.lean,Mathlib/Analysis/Complex/Positivity.lean,Mathlib/Analysis/Complex/Schwarz.lean,Mathlib/Analysis/Complex/UnitDisc/Basic.lean,Mathlib/Analysis/Complex/UpperHalfPlane/Exp.lean,Mathlib/Analysis/Complex/UpperHalfPlane/Metric.lean,Mathlib/Analysis/Fourier/AddCircle.lean,Mathlib/Analysis/Fourier/AddCircleMulti.lean,Mathlib/Analysis/Fourier/FourierTransformDeriv.lean,Mathlib/Analysis/Fourier/Inversion.lean,Mathlib/Analysis/Fourier/PoissonSummation.lean,Mathlib/Analysis/InnerProductSpace/TwoDim.lean,Mathlib/Analysis/MellinTransform.lean,Mathlib/Analysis/Normed/Group/Continuity.lean,Mathlib/Analysis/Normed/Lp/WithLp.lean,Mathlib/Analysis/PSeries.lean,Mathlib/Analysis/PSeriesComplex.lean,Mathlib/Analysis/SpecialFunctions/CompareExp.lean,Mathlib/Analysis/SpecialFunctions/Complex/Arctan.lean,Mathlib/Analysis/SpecialFunctions/Complex/Arg.lean,Mathlib/Analysis/SpecialFunctions/Complex/Circle.lean,Mathlib/Analysis/SpecialFunctions/Complex/Log.lean,Mathlib/Analysis/SpecialFunctions/Complex/LogBounds.lean,Mathlib/Analysis/SpecialFunctions/Exp.lean,Mathlib/Analysis/SpecialFunctions/Exponential.lean,Mathlib/Analysis/SpecialFunctions/Gamma/Basic.lean,Mathlib/Analysis/SpecialFunctions/Gamma/Beta.lean,Mathlib/Analysis/SpecialFunctions/Gamma/Deriv.lean,Mathlib/Analysis/SpecialFunctions/Gaussian/FourierTransform.lean,Mathlib/Analysis/SpecialFunctions/Gaussian/GaussianIntegral.lean,Mathlib/Analysis/SpecialFunctions/Gaussian/PoissonSummation.lean,Mathlib/Analysis/SpecialFunctions/ImproperIntegrals.lean,Mathlib/Analysis/SpecialFunctions/Integrals.lean,Mathlib/Analysis/SpecialFunctions/Log/Summable.lean,Mathlib/Analysis/SpecialFunctions/PolarCoord.lean,Mathlib/Analysis/SpecialFunctions/Pow/Asymptotics.lean,Mathlib/Analysis/SpecialFunctions/Pow/Continuity.lean,Mathlib/Analysis/SpecialFunctions/Pow/Deriv.lean,Mathlib/Analysis/SpecialFunctions/Pow/Real.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/ArctanDeriv.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Basic.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/ComplexDeriv.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Cotangent.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Series.lean,Mathlib/CategoryTheory/Abelian/FreydMitchell.lean,Mathlib/CategoryTheory/Abelian/GrothendieckAxioms/Connected.lean,Mathlib/CategoryTheory/Abelian/GrothendieckAxioms/Indization.lean,Mathlib/CategoryTheory/Abelian/GrothendieckCategory/Coseparator.lean 205 10 ['Champitoad', 'github-actions', 'joelriou'] nobody
103-83762
3 months ago
103-85035
3 months ago
0-38059
10 hours
20454 urkud
author:urkud
chore(TangentCone): review names Also add some `@[simp]` attrs. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis merge-conflict 201/139 Mathlib/Analysis/Analytic/IteratedFDeriv.lean,Mathlib/Analysis/Calculus/ContDiff/Basic.lean,Mathlib/Analysis/Calculus/ContDiff/Bounds.lean,Mathlib/Analysis/Calculus/ContDiff/Defs.lean,Mathlib/Analysis/Calculus/ContDiff/FTaylorSeries.lean,Mathlib/Analysis/Calculus/Deriv/Abs.lean,Mathlib/Analysis/Calculus/Deriv/Basic.lean,Mathlib/Analysis/Calculus/FDeriv/Add.lean,Mathlib/Analysis/Calculus/FDeriv/Basic.lean,Mathlib/Analysis/Calculus/FDeriv/Equiv.lean,Mathlib/Analysis/Calculus/FDeriv/Measurable.lean,Mathlib/Analysis/Calculus/FDeriv/RestrictScalars.lean,Mathlib/Analysis/Calculus/FDeriv/Symmetric.lean,Mathlib/Analysis/Calculus/IteratedDeriv/Lemmas.lean,Mathlib/Analysis/Calculus/MeanValue.lean,Mathlib/Analysis/Calculus/TangentCone.lean,Mathlib/Analysis/Calculus/Taylor.lean,Mathlib/Analysis/Calculus/VectorField.lean,Mathlib/Analysis/Convex/SpecificFunctions/Deriv.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/InverseDeriv.lean,Mathlib/Geometry/Manifold/Instances/Real.lean,Mathlib/Geometry/Manifold/IsManifold/Basic.lean,Mathlib/Geometry/Manifold/MFDeriv/UniqueDifferential.lean,Mathlib/Geometry/Manifold/VectorBundle/Tangent.lean,Mathlib/MeasureTheory/Integral/FundThmCalculus.lean 25 3 ['github-actions', 'sgouezel', 'urkud'] nobody
103-42843
3 months ago
103-42843
3 months ago
12-11675
12 days
14760 FR-vdash-bot
author:FR-vdash-bot
feat: define `IGame` --- - [ ] depends on: #7162 [diff](https://github.com/leanprover-community/mathlib4/compare/FR_game_relabelling..FR_igame) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-logic merge-conflict WIP 1427/661 Mathlib.lean,Mathlib/SetTheory/Game/Basic.lean,Mathlib/SetTheory/Game/Birthday.lean,Mathlib/SetTheory/Game/IGame.lean,Mathlib/SetTheory/Game/Impartial.lean,Mathlib/SetTheory/Game/Nim.lean,Mathlib/SetTheory/Game/Ordinal.lean,Mathlib/SetTheory/Game/PGame.lean,Mathlib/SetTheory/Game/Relabelling.lean,Mathlib/SetTheory/Game/Short.lean,Mathlib/SetTheory/Surreal/Basic.lean,scripts/style-exceptions.txt 12 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
103-39674
3 months ago
103-39677
3 months ago
0-1038
17 minutes
21608 JLimperg
author:JLimperg
Aesop forward benchmark: forward no-precomp rpinf pr-release Not a real PR, just for benchmarking. merge-conflict 38/29 Mathlib/Data/List/InsertIdx.lean,Mathlib/Data/Nat/Prime/Defs.lean,Mathlib/Tactic/Recall.lean,Mathlib/Topology/List.lean,Test.lean,lake-manifest.json,lakefile.lean,lean-toolchain 8 13 ['JLimperg', 'github-actions', 'leanprover-bot'] nobody
103-17576
3 months ago
120-11640
4 months ago*
0-0
0 seconds*
21609 JLimperg
author:JLimperg
Aesop forward benchmark: forward no-precomp Not a real PR, just for benchmarking. merge-conflict 38/29 Mathlib/Data/List/InsertIdx.lean,Mathlib/Data/Nat/Prime/Defs.lean,Mathlib/Tactic/Recall.lean,Mathlib/Topology/List.lean,Test.lean,lake-manifest.json,lakefile.lean,lean-toolchain 8 13 ['JLimperg', 'github-actions', 'leanprover-bot'] nobody
103-15940
3 months ago
120-11504
4 months ago*
0-0
0 seconds*
16550 awainverse
author:awainverse
feat(ModelTheory): A typeclass for languages expanding other languages Defines `L.Expands L'` to consist of a privileged injective inclusion, `L'.Inclusion L`, from `L'` to `L`, corresponding to one language being a subset of the other in set-theoretic foundations. Replaces `L.IsOrdered` with `L.Expands Language.order` and `L.OrderLHom` with `Language.order.Inclusion L` Redefines `leSymb` in terms of `Language.order.Inclusion L` Deletions: - `FirstOrder.Language.IsOrdered` - `FirstOrder.Language.OrderLHom` - `instance : IsOrdered Language.order` - `sum.instIsOrdered` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-logic merge-conflict awaiting-author 97/43 Mathlib/ModelTheory/LanguageMap.lean,Mathlib/ModelTheory/Order.lean 2 9 ['YaelDillies', 'awainverse', 'github-actions'] nobody
102-81711
3 months ago
102-81712
3 months ago
0-61590
17 hours
13686 fpvandoorn
author:fpvandoorn
feat: some finset lemmas * From the Sobolev inequality project * The increase in imports in `Mathlib.Data.Finset.Update` is not problematic: it is only imported in MeasureTheory files. Co-authored-by: Heather Macbeth 25316162+hrmacbeth@users.noreply.github.com --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data merge-conflict awaiting-author 69/7 Mathlib/Data/Finset/Basic.lean,Mathlib/Data/Finset/Lattice/Lemmas.lean,Mathlib/Data/Finset/Update.lean 3 7 ['YaelDillies', 'fpvandoorn', 'github-actions', 'urkud'] nobody
101-81342
3 months ago
101-81342
3 months ago
98-49006
98 days
14313 grhkm21
author:grhkm21
feat(RepresentationTheory/FdRep): FdRep is a full subcategory of Rep ``` /-- Equivalence between `FDRep` and the full subcategory of finite dimensional `Rep`. -/ def equivFiniteDimensional : FDRep k G ≌ FullSubcategory (fun V : Rep k G ↦ FiniteDimensional k V) ``` new-contributor t-algebra t-category-theory merge-conflict
label:t-algebra$
47/8 Mathlib/RepresentationTheory/FDRep.lean 1 19 ['github-actions', 'grhkm21', 'joelriou', 'kim-em', 'mathlib-bors'] nobody
101-29873
3 months ago
101-29873
3 months ago
125-12755
125 days
22331 jjdishere
author:jjdishere
feat(RingTheory/Perfectoid): define integral perfectoid rings In this PR, we define the integral perfectoid ring and the perfectoid pseudo uniformizers. --- - [ ] depends on: #21564 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-number-theory merge-conflict blocked-by-other-PR WIP
label:t-algebra$
1099/15 Mathlib.lean,Mathlib/Algebra/Ring/Aut.lean,Mathlib/FieldTheory/Perfect.lean,Mathlib/RingTheory/AdicCompletion/Basic.lean,Mathlib/RingTheory/Ideal/Maps.lean,Mathlib/RingTheory/Ideal/Quotient/Defs.lean,Mathlib/RingTheory/Ideal/Quotient/PowTransition.lean,Mathlib/RingTheory/Perfection.lean,Mathlib/RingTheory/Perfectoid/BDeRham.lean,Mathlib/RingTheory/Perfectoid/FontaineTheta.lean,Mathlib/RingTheory/Perfectoid/IntergalPerfectoid.lean,Mathlib/RingTheory/Perfectoid/Untilt.lean,Mathlib/RingTheory/WittVector/Basic.lean,Mathlib/RingTheory/WittVector/Complete.lean,Mathlib/RingTheory/WittVector/TeichmullerSeries.lean,docs/references.bib 16 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
100-21658
3 months ago
100-21658
3 months ago
0-0
0 seconds
22332 jjdishere
author:jjdishere
feat(RingTheory/Perfectoid): Fontaine's theta map is surjective In this PR, we show that Fontaine's theta map is surjective. --- - [ ] depends on: #21564 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-number-theory merge-conflict blocked-by-other-PR WIP
label:t-algebra$
1127/15 Mathlib.lean,Mathlib/Algebra/Ring/Aut.lean,Mathlib/FieldTheory/Perfect.lean,Mathlib/RingTheory/AdicCompletion/Basic.lean,Mathlib/RingTheory/Ideal/Maps.lean,Mathlib/RingTheory/Ideal/Quotient/Defs.lean,Mathlib/RingTheory/Ideal/Quotient/PowTransition.lean,Mathlib/RingTheory/Perfection.lean,Mathlib/RingTheory/Perfectoid/BDeRham.lean,Mathlib/RingTheory/Perfectoid/FontaineTheta.lean,Mathlib/RingTheory/Perfectoid/Untilt.lean,Mathlib/RingTheory/WittVector/Basic.lean,Mathlib/RingTheory/WittVector/Complete.lean,Mathlib/RingTheory/WittVector/TeichmullerSeries.lean,docs/references.bib 15 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
100-21657
3 months ago
100-21657
3 months ago
0-37
37 seconds
18626 hannahfechtner
author:hannahfechtner
feat : define Artin braid groups Define the Artin braid group on infinitely many strands. Includes a toGroup function which defines a function out of the braid group to any other group (given a function which satisfies the braid relations) (more to come in this file; next up: Artin braid groups on finitely many strands) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra merge-conflict awaiting-author
label:t-algebra$
91/0 Mathlib.lean,Mathlib/GroupTheory/SpecificGroups/BraidGroup/Basic.lean 2 22 ['github-actions', 'hannahfechtner', 'jcommelin', 'joelriou'] nobody
100-14184
3 months ago
100-14184
3 months ago
15-40648
15 days
10823 alexkeizer
author:alexkeizer
feat: convert curried type functions into uncurried type functions Adds a conversion `TypeFun.ofCurried : CurriedTypeFun.{u, v} n -> TypeFun.{u, v} n`, where `CurriedTypeFun.{u,v} n` is a (def-eq) abbreviation for `Type u -> ... -> Type u -> Type v`, i.e., the type of *curried* functions taking `n` arguments of type `Type u` to return an element of `Type v`, and `TypeFun.{u, v} n` is an abbreviation for `TypeVec.{u} n -> Type v`. It is generally more idiomatic to define type functions with multiple arguments in the curried style, but in the QPF development we use the uncurried equivalent `TypeVec n -> Type _`. Thus, having a canonical conversion from curried functions to uncurried gives us a canonical way to ask if a curried type function, say `Sum` is a QPF (namely, "is there an instance of `MvQPF (TypeFun.ofCurried Sum)`"). --- This is code ported from https://github.com/alexkeizer/QpfTypes, where this conversion is crucial in presenting a high-level interface, in terms of idiomatic, curried, type functions to users, while being built on QPFs (and thus, uncurried typefunctions) underneath. There is also a conversion in the other direction, from uncurried to curried, which I've decided to PR later, to keep this PR smaller and hopefully easier to review. - [x] depends on: #10818 (all changes to `Fin2.lean` are part of 10818, not the current PR) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data merge-conflict awaiting-author 66/0 Mathlib.lean,Mathlib/Data/TypeFun.lean 2 9 ['YaelDillies', 'alexkeizer', 'github-actions', 'leanprover-community-mathlib4-bot'] nobody
100-7904
3 months ago
unknown
unknown
13648 urkud
author:urkud
feat(Topology/Module): generalize `ContinuousLinearMap.compSL` Generalize `ContinuousLinearMap.compSL` to topological vector spaces. --- - [ ] depends on: #15217 This PR is not polished yet, but the main statement is there. @ADedecker This answers a question I asked you on Zulip a few months ago. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-analysis t-topology merge-conflict awaiting-author
label:t-algebra$
23/18 Mathlib/Analysis/NormedSpace/OperatorNorm/Bilinear.lean,Mathlib/Topology/Algebra/Module/StrongTopology.lean 2 5 ['fpvandoorn', 'github-actions', 'mathlib4-dependent-issues-bot', 'urkud'] nobody
98-30994
3 months ago
98-30994
3 months ago
0-0
0 seconds
19372 Command-Master
author:Command-Master
find defeq abuse using diagnostics --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) - [ ] depends on: #19177 large-import merge-conflict blocked-by-other-PR 169/1 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter.lean,Mathlib/Tactic/Linter/FindDefEqAbuse.lean,MathlibTest/FindDefEqAbuse.lean,lakefile.lean 6 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
98-30494
3 months ago
98-30494
3 months ago
0-0
0 seconds
21684 mattrobball
author:mattrobball
draft merge-conflict 13/11 Mathlib/CategoryTheory/Category/Cat/AsSmall.lean,Mathlib/CategoryTheory/Closed/FunctorToTypes.lean,Mathlib/CategoryTheory/Closed/Types.lean,Mathlib/FieldTheory/IsAlgClosed/Classification.lean,Mathlib/SetTheory/Ordinal/Basic.lean,Mathlib/Topology/Category/LightProfinite/Basic.lean,lean-toolchain 7 4 ['github-actions', 'leanprover-bot', 'mattrobball'] nobody
98-24564
3 months ago
98-24564
3 months ago
0-0
0 seconds
21722 mattrobball
author:mattrobball
test merge-conflict 76/23 Mathlib/CategoryTheory/Category/Cat/AsSmall.lean,Mathlib/CategoryTheory/Closed/FunctorToTypes.lean,Mathlib/CategoryTheory/Closed/Types.lean,Mathlib/FieldTheory/IsAlgClosed/Classification.lean,Mathlib/Order/Hom/Lattice.lean,Mathlib/SetTheory/Ordinal/Basic.lean,Mathlib/Topology/Category/LightProfinite/Basic.lean,lean-toolchain,scratch.lean 9 4 ['github-actions', 'leanprover-bot', 'mattrobball'] nobody
98-24563
3 months ago
98-24563
3 months ago
0-0
0 seconds
22408 JLimperg
author:JLimperg
Aesop forward bench: precomp only rpinf --- Not a real PR (yet), just for benchmarking. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) dependency-bump merge-conflict 5/3 lake-manifest.json,lakefile.lean,scripts/bench/fake-root/lib/lean/libleanshared.so,scripts/bench/run 4 6 ['JLimperg', 'github-actions', 'leanprover-bot'] nobody
98-19398
3 months ago
98-19398
3 months ago
0-0
0 seconds
13964 pechersky
author:pechersky
feat(Data/DigitExpansion): begin defining variant of reals without rationals Based on a de Bruijn 1976 paper. This file is just the basic definition of a digit expansion. Will be followed up with furhter constructions. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data merge-conflict 518/0 Mathlib.lean,Mathlib/Data/DigitExpansion/Defs.lean,docs/references.bib 3 11 ['eric-wieser', 'github-actions', 'kim-em', 'pechersky'] dupuisf
assignee:dupuisf
98-15949
3 months ago
225-32457
7 months ago
129-57991
129 days
21339 vihdzp
author:vihdzp
fix(Data/List/Lex): remove duplicate `List.LE` instance Mathlib currently duplicates the Lean core instance for `≤` in lists in an incompatible way. We delete this duplicate instance. See [Zulip](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Two.20.60List.2ELE.60.20instances.3F/near/497241115). --- This is a very quick and dirty fix. Core Lean provides all of the theorems we need to prove `≤` forms a linear order, but it provides them in terms of `Std` relation typeclasses which currently see no use in Mathlib. I've added the instances that were required to get the list theorems working. In the future, we really ought to unify the core and Mathlib relation typeclasses. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data merge-conflict 24/22 Mathlib/Data/List/Lex.lean,Mathlib/Data/String/Basic.lean,Mathlib/Topology/Category/Profinite/Nobeling.lean 3 1 ['github-actions'] nobody
98-11736
3 months ago
98-11736
3 months ago
16-65973
16 days
11212 shuxuezhuyi
author:shuxuezhuyi
feat(GroupTheory/GroupAction): instance `MulAction (β ⧸ H) α` We instance this naturally from `MulAction β α` when `H` is a normal subgroup and acts trivially on `α`. We also instance `IsometricSMul (M ⧸ N) X` in this way. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-algebra merge-conflict awaiting-author
label:t-algebra$
53/1 Mathlib/GroupTheory/GroupAction/Quotient.lean,Mathlib/Topology/MetricSpace/IsometricSMul.lean 2 6 ['YaelDillies', 'github-actions', 'grunweg', 'urkud'] eric-wieser
assignee:eric-wieser
98-5719
3 months ago
98-5719
3 months ago
193-70524
193 days
14060 YnirPaz
author:YnirPaz
feat(SetTheory/Ordinal/Clubs): define club sets and prove basic properties Create a file where club sets are defined and their basic properties are proven. I also created a new recursion principle for ordinals, bounded recursion. --- - [ ] depends on: #19189 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-logic merge-conflict blocked-by-other-PR 315/3 Mathlib.lean,Mathlib/Order/SuccPred/Limit.lean,Mathlib/SetTheory/Cardinal/Cofinality.lean,Mathlib/SetTheory/Ordinal/Arithmetic.lean,Mathlib/SetTheory/Ordinal/Club.lean,Mathlib/SetTheory/Ordinal/Topology.lean 6 93 ['YaelDillies', 'YnirPaz', 'alreadydone', 'dupuisf', 'github-actions', 'mathlib4-dependent-issues-bot', 'vihdzp', 'zeramorphic'] nobody
97-58697
3 months ago
97-58697
3 months ago
92-44198
92 days
16837 vihdzp
author:vihdzp
feat(Data/List/SplitBy): characterization of `List.splitBy` --- - [x] depends on: #16818 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data merge-conflict awaiting-author 151/9 Mathlib/Data/List/Flatten.lean,Mathlib/Data/List/SplitBy.lean 2 13 ['YaelDillies', 'github-actions', 'mathlib4-dependent-issues-bot', 'vihdzp'] nobody
97-58451
3 months ago
97-58451
3 months ago
9-85039
9 days
16421 FR-vdash-bot
author:FR-vdash-bot
feat: `QuotLike` This typeclass is primarily for use by type synonyms of `Quot` and `Quotient`. Using `QuotLike` API for type synonyms of `Quot` and `Quotient` will avoid defeq abuse caused by directly using `Quot` and `Quotient` APIs. --- Some of the naming may need to be discussed. For example, `⟦·⟧` is currently called `mkQ` in names. This distinguishes it from other `.mk`s and makes it possible to write the quotient map as `mkQ` `mkQ'` `mkQ_ h`. But this will also require changing the old lemma names. [Zulip](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/migrate.20to.20.60QuotLike.60.20API) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data RFC merge-conflict awaiting-author 735/1 Mathlib.lean,Mathlib/Data/QuotLike.lean,Mathlib/Logic/Relation.lean,test/QuotLike.lean 4 7 ['FR-vdash-bot', 'YaelDillies', 'github-actions', 'urkud'] nobody
97-58451
3 months ago
97-58451
3 months ago
58-8650
58 days
17105 vihdzp
author:vihdzp
feat(Data/List/RunLength): run-length encoding We define the run-length encoding of a list. We provide a basic API, as well as a recursion principle. --- - [ ] depends on: #16837 - [x] depends on: #17106 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data merge-conflict blocked-by-other-PR 286/1 Mathlib/Data/List/Flatten.lean,Mathlib/Data/List/RunLength.lean,Mathlib/Data/List/SplitBy.lean 3 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
97-58450
3 months ago
97-58450
3 months ago
0-0
0 seconds
19700 vihdzp
author:vihdzp
chore(SetTheory/Ordinal/Basic): tweak `type r = 0`, `type r = 1`, etc. lemmas We give shorter names to these lemmas (e.g. `type_eq_zero` instead of `type_eq_zero_of_empty`), and deprecate a bunch of duplicates. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-set-theory awaiting-CI merge-conflict 51/38 Mathlib/SetTheory/Ordinal/Basic.lean 1 1 ['github-actions'] nobody
97-58204
3 months ago
97-58204
3 months ago
0-0
0 seconds
22340 sinhp
author:sinhp
feat(CategoryTheory): Locally Cartesian Closed Categories (Beck-Chevalley Conditions) Building on top of the API of `ExponentiableMorphism` in #22321, we state and prove Beck-Chevalley conditions. This will be crucial for our development of polynomial functors along exponentiable morphisms. Co-authored-by: Emily Riehl --- - [ ] depends on: #22321 - [ ] depends on: #22319 - [ ] depends on: #21525 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-category-theory merge-conflict blocked-by-other-PR WIP 1144/24 Mathlib.lean,Mathlib/CategoryTheory/Comma/Over/Basic.lean,Mathlib/CategoryTheory/Comma/Over/Pullback.lean,Mathlib/CategoryTheory/Comma/Over/Sections.lean,Mathlib/CategoryTheory/Galois/Examples.lean,Mathlib/CategoryTheory/LocallyCartesianClosed/Basic.lean,Mathlib/CategoryTheory/LocallyCartesianClosed/BeckChevalley.lean,docs/references.bib 8 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
96-19545
3 months ago
96-19545
3 months ago
0-17
17 seconds
21959 BGuillemet
author:BGuillemet
feat(Topology/ContinuousMap): Stone-Weierstrass theorem for MvPolynomial Add the subalgebra of multivariate polynomials and prove it separates points, on the same model as `ContinuousMap/Polynomial.lean`. Prove the Stone-Weierstrass theorem and some variations for multivariate polynomials. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-topology merge-conflict 285/1 Mathlib.lean,Mathlib/Topology/ContinuousMap/MvPolynomial.lean,Mathlib/Topology/ContinuousMap/StoneWeierstrass.lean 3 1 ['github-actions'] nobody
96-15887
3 months ago
96-15887
3 months ago
16-76141
16 days
22532 jcommelin
author:jcommelin
chore(RingTheory/TensorProduct): cleanup --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict WIP
label:t-algebra$
68/28 Mathlib/RingTheory/Finiteness/TensorProduct.lean,Mathlib/RingTheory/TensorProduct/Adjoin.lean,Mathlib/RingTheory/TensorProduct/Basic.lean,Mathlib/RingTheory/TensorProduct/Finite.lean 4 1 ['github-actions'] nobody
96-11182
3 months ago
96-11182
3 months ago
0-31
31 seconds
21275 joneugster
author:joneugster
feat(Cache): decompress downloaded files directly Extract downloaded files directly. This increases parallelism as files are downloaded in parallel and downloading/decompressing use different hardware (network/cpu) --- - [ ] depends on: #21238 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) CI t-meta merge-conflict blocked-by-other-PR WIP 66/15 Cache/IO.lean,Cache/Lean.lean,Cache/Requests.lean 3 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
94-34141
3 months ago
94-34141
3 months ago
0-0
0 seconds
19177 adomani
author:adomani
test: the findDefEqAbuse linter This is a prototype, as per [this Zulip discussion](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Locating.20defeq.20abuse) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import merge-conflict 126/0 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter.lean,Mathlib/Tactic/Linter/FindDefEqAbuse.lean,MathlibTest/FindDefEqAbuse.lean 5 1 ['github-actions'] nobody
94-17900
3 months ago
94-17900
3 months ago
0-0
0 seconds
20750 adomani
author:adomani
feat: the envLinter syntax linter The `envLinter` syntax linter emits a warning at the end of a file if `#lint` reports an error. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-linter merge-conflict 69/0 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter.lean,Mathlib/Tactic/Linter/EnvLinter.lean,MathlibTest/EnvLinter.lean 5 15 ['adomani', 'github-actions', 'grunweg'] nobody
94-17654
3 months ago
94-17654
3 months ago
51-71438
51 days
22359 adomani
author:adomani
feat(whitespace): do not allow indented doc-strings In a doc-string, Do not allow the first character after the first line break to be a space. --- There are approximately 2.5k exceptions. I think that they should be unindented, judging from the sample that I looked at, but won't act on it, unless there is a clear plan to fix and merge this modification! --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-linter merge-conflict WIP 222/70 Archive/Wiedijk100Theorems/BuffonsNeedle.lean,Mathlib.lean,Mathlib/Algebra/Module/SpanRank.lean,Mathlib/AlgebraicTopology/SimplicialSet/NerveAdjunction.lean,Mathlib/Analysis/Asymptotics/ExpGrowth.lean,Mathlib/Data/Matroid/Circuit.lean,Mathlib/Init.lean,Mathlib/Lean/Meta/RefinedDiscrTree/Encode.lean,Mathlib/LinearAlgebra/Dimension/StrongRankCondition.lean,Mathlib/LinearAlgebra/LinearIndependent/Basic.lean,Mathlib/LinearAlgebra/LinearIndependent/Defs.lean,Mathlib/Tactic.lean,Mathlib/Tactic/FunProp/Decl.lean,Mathlib/Tactic/FunProp/Theorems.lean,Mathlib/Tactic/Linter.lean,Mathlib/Tactic/Linter/DocString.lean,Mathlib/Topology/Path.lean,Mathlib/Topology/UnitInterval.lean,MathlibTest/LintDocstring.lean,lakefile.lean 20 1 ['github-actions'] nobody
94-16819
3 months ago
94-16819
3 months ago
0-0
0 seconds
20267 joelriou
author:joelriou
feat(CategoryTheory): comma categories are accessible --- (I shall probably not work on this PR in the near future.) - [ ] depends on: #19937 - [ ] depends on: #19945 - [ ] depends on: #19959 - [ ] depends on: #20005 - [ ] depends on: #19955 - [ ] depends on: #20263 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory merge-conflict awaiting-author blocked-by-other-PR WIP 1513/7 Mathlib.lean,Mathlib/CategoryTheory/Comma/Arrow.lean,Mathlib/CategoryTheory/Comma/CardinalArrow.lean,Mathlib/CategoryTheory/EssentiallySmall.lean,Mathlib/CategoryTheory/Limits/Comma.lean,Mathlib/CategoryTheory/Limits/TypesFiltered.lean,Mathlib/CategoryTheory/Presentable/Basic.lean,Mathlib/CategoryTheory/Presentable/CardinalFilteredPresentation.lean,Mathlib/CategoryTheory/Presentable/Comma.lean,Mathlib/CategoryTheory/Presentable/IsCardinalFiltered.lean,Mathlib/CategoryTheory/Presentable/Limits.lean,Mathlib/CategoryTheory/Presentable/LocallyPresentable.lean,Mathlib/CategoryTheory/Presentable/ParallelMaps.lean,Mathlib/SetTheory/Cardinal/HasCardinalLT.lean,docs/references.bib 15 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
92-1122
3 months ago
147-30236
4 months ago
0-0
0 seconds
18470 FR-vdash-bot
author:FR-vdash-bot
perf: lower the priority of `Normed*.to*` instances --- From #7873. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) slow-typeclass-synthesis t-algebra t-analysis merge-conflict
label:t-algebra$
28/0 Mathlib/Analysis/Normed/Field/Basic.lean,Mathlib/Analysis/Normed/Group/Basic.lean 2 9 ['FR-vdash-bot', 'github-actions', 'jcommelin', 'leanprover-bot'] nobody
91-73714
2 months ago
91-73714
2 months ago
130-5197
130 days
22538 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 - [ ] depends on: #22531 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis merge-conflict blocked-by-other-PR 228/8 Mathlib.lean,Mathlib/Algebra/BigOperators/Ring/List.lean,Mathlib/Analysis/Analytic/Basic.lean,Mathlib/Analysis/Analytic/Binomial.lean,Mathlib/Analysis/Calculus/FormalMultilinearSeries.lean,Mathlib/RingTheory/Binomial.lean,scripts/noshake.json 7 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
90-80019
2 months ago
90-80019
2 months ago
0-1173
19 minutes
16944 YnirPaz
author:YnirPaz
feat(SetTheory/Cardinal/Cofinality): lemmas about limit ordinals and cofinality Prove that a singular cardinal has a limit aleph index and that a limit ordinal and positive cofinality. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-set-theory merge-conflict WIP 18/0 Mathlib/SetTheory/Cardinal/Cofinality.lean 1 8 ['YnirPaz', 'github-actions', 'vihdzp'] nobody
90-66590
2 months ago
90-66590
2 months ago
1-84890
1 day
17368 Felix-Weilacher
author:Felix-Weilacher
feat(Topology/Baire/BaireMeasurable): add the Kuratowski-Ulam theorem Add the Kuratowski-Ulam theorem, which one can think of as a "Fubini" for Baire category. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology merge-conflict 187/1 Mathlib/MeasureTheory/MeasurableSpace/Basic.lean,Mathlib/Order/Filter/Basic.lean,Mathlib/Topology/Baire/BaireMeasurable.lean,Mathlib/Topology/Constructions.lean,Mathlib/Topology/GDelta/Basic.lean 5 6 ['Felix-Weilacher', 'github-actions', 'urkud'] nobody
90-11383
2 months ago
90-11383
2 months ago
72-13986
72 days
8767 eric-wieser
author:eric-wieser
refactor(Cache): tidy lake-manifest parsing in Cache This now respects local copies of Mathlib dependencies (though in practice these invalidate the *online* cache because to point to local copies of Mathlib, the hash for `lakefile.lean` and `lake-manifest.json` is first invalidated). --- - [x] depends on: #11492 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta merge-conflict 49/49 Cache/Hashing.lean,Cache/IO.lean,lake-manifest.json 3 8 ['digama0', 'eric-wieser', 'github-actions', 'leanprover-community-mathlib4-bot'] nobody
88-73446
2 months ago
270-39396
8 months ago
119-35643
119 days
22434 qawbecrdtey
author:qawbecrdtey
feat(Mathlib/Analysis/Normed/Lp/WithLp): Added more instances for `WithLp` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis merge-conflict awaiting-author 51/22 Mathlib/Analysis/Normed/Lp/WithLp.lean 1 11 ['eric-wieser', 'github-actions', 'leanprover-bot', 'qawbecrdtey'] nobody
88-16485
2 months ago
88-16485
2 months ago
1-79072
1 day
15578 znssong
author:znssong
feat(Function): Fixed points of function `f` with `f(x) >= x` We added some lemmas of fixed points of function `f` with `f(x) >= x`, where `f : α → α` is a function on a finite type `α`. This will be needed in proof of Bondy-Chvátal theorem. --- See also branch `meow-sister/BondyChvatal`. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-analysis merge-conflict awaiting-author 82/0 Mathlib.lean,Mathlib/Dynamics/FixedPoints/Basic.lean,Mathlib/Dynamics/FixedPoints/Increasing.lean 3 32 ['Ruben-VandeVelde', 'YaelDillies', 'github-actions', 'urkud', 'vihdzp', 'znssong'] nobody
88-11713
2 months ago
88-11713
2 months ago
29-48368
29 days
8793 101damnations
author:101damnations
feat(RepresentationTheory/GroupCohomology/Hilbert90): add Hilbert's original theorem 90 --- This PR proves that given a finite cyclic Galois extension $L/K,$ a generator $g \in Gal(L/K),$ and an element `x : L` such that $N_{L/K}(x) = 1,$ there exists `y : L` such that $g(y)/y = x.$ It's a direct proof instead of analysing the cohomology of finite cyclic groups in general, but I'm hoping the API should still be useful for/alongside that. - [x] depends on: #8785 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict awaiting-author
label:t-algebra$
213/11 Mathlib/GroupTheory/OrderOfElement.lean,Mathlib/RepresentationTheory/GroupCohomology/Hilbert90.lean,Mathlib/RepresentationTheory/GroupCohomology/LowDegree.lean,Mathlib/RepresentationTheory/Rep.lean 4 3 ['github-actions', 'joelriou', 'leanprover-community-mathlib4-bot'] nobody
87-57302
2 months ago
87-57303
2 months ago
0-0
0 seconds
22517 j-loreaux
author:j-loreaux
feat: `ℕ+` powers in semigroups --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import merge-conflict WIP 275/28 Mathlib.lean,Mathlib/Algebra/Group/Defs.lean,Mathlib/Algebra/Group/Ext.lean,Mathlib/Algebra/Group/PNatPowAssoc.lean,Mathlib/Algebra/Group/PPow.lean,Mathlib/Algebra/Group/TypeTags/Basic.lean,Mathlib/Algebra/Ring/Ext.lean,Mathlib/Algebra/Ring/ULift.lean,Mathlib/Data/Num/Lemmas.lean,Mathlib/Data/Real/Basic.lean,Mathlib/Data/ZMod/Defs.lean,Mathlib/LinearAlgebra/LinearPMap.lean,Mathlib/NumberTheory/Dioph.lean,Mathlib/Tactic/ToAdditive/Frontend.lean 14 4 ['github-actions', 'j-loreaux', 'leanprover-bot'] nobody
87-46309
2 months ago
87-46310
2 months ago
0-27
27 seconds
22805 ScottCarnahan
author:ScottCarnahan
feat (FieldTheory/Finite): fixed points of frobenius This PR identifies the prime field with the fixed points of frobenius. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict WIP
label:t-algebra$
325/7 Mathlib/Algebra/Algebra/ZMod.lean,Mathlib/Algebra/Field/Subfield/Basic.lean,Mathlib/FieldTheory/Finite/Basic.lean,Mathlib/FieldTheory/Finite/GaloisField.lean 4 1 ['github-actions'] nobody
86-22425
2 months ago
86-22425
2 months ago
0-0
0 seconds
22660 Ruben-VandeVelde
author:Ruben-VandeVelde
chore: follow naming convention around Group.IsNilpotent --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict
label:t-algebra$
133/67 Mathlib/GroupTheory/Frattini.lean,Mathlib/GroupTheory/Nilpotent.lean,Mathlib/GroupTheory/SpecificGroups/ZGroup.lean 3 1 ['github-actions'] nobody
84-38142
2 months ago
84-38142
2 months ago
10-48025
10 days
20424 erdOne
author:erdOne
feat(RingTheory): evaluation of power series --- - [ ] depends on: #20425 - [x] depends on: #20426 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict
label:t-algebra$
425/8 Mathlib.lean,Mathlib/RingTheory/AdicCompletion/Noetherian.lean,Mathlib/RingTheory/Filtration.lean,Mathlib/RingTheory/PowerSeries/Basic.lean,Mathlib/RingTheory/PowerSeries/Eval.lean,Mathlib/RingTheory/PowerSeries/Trunc.lean 6 11 ['AntoineChambert-Loir', 'alreadydone', 'erdOne', 'eric-wieser', 'github-actions', 'mathlib4-dependent-issues-bot'] nobody
84-16605
2 months ago
118-83953
3 months ago
0-3944
1 hour
21564 jjdishere
author:jjdishere
feat(RingTheory/Perfectoid): Fontaine's theta map and the de Rham period rings In this PR, we define the Fontaine's theta map and the peroid ring B_dR. --- - [x] depends on: #21563 [untilt map] - [ ] depends on: #21582 - [ ] depends on: #22320 - [ ] depends on: #22330 [which depends on the previous one] [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-number-theory merge-conflict blocked-by-other-PR
label:t-algebra$
1044/15 Mathlib.lean,Mathlib/Algebra/Ring/Aut.lean,Mathlib/FieldTheory/Perfect.lean,Mathlib/RingTheory/AdicCompletion/Basic.lean,Mathlib/RingTheory/Ideal/Maps.lean,Mathlib/RingTheory/Ideal/Quotient/Defs.lean,Mathlib/RingTheory/Ideal/Quotient/PowTransition.lean,Mathlib/RingTheory/Perfection.lean,Mathlib/RingTheory/Perfectoid/BDeRham.lean,Mathlib/RingTheory/Perfectoid/FontaineTheta.lean,Mathlib/RingTheory/Perfectoid/Untilt.lean,Mathlib/RingTheory/WittVector/Basic.lean,Mathlib/RingTheory/WittVector/Complete.lean,Mathlib/RingTheory/WittVector/TeichmullerSeries.lean,docs/references.bib 15 5 ['AntoineChambert-Loir', 'github-actions', 'jjdishere', 'mathlib4-dependent-issues-bot'] riccardobrasca
assignee:riccardobrasca
84-13221
2 months ago
100-22411
3 months ago
0-0
0 seconds
13999 adomani
author:adomani
feat: a linter to flag potential confusing conventions Currently, the linter flags all uses of * `a - b` where `a b : Nat`; * `a / b` where `a b : Nat` or `a b : Int`; * `a / 0` more or less whenever the type of `a` has a `0` and a division. This comes up often when starting to use Lean and hopefully the flag can help mitigate initial confusions. When the local context contains the relevant inequality/divisibility hypothesis, the linter is quiet. A recent [Zulip discussion](https://leanprover.zulipchat.com/#narrow/stream/113489-new-members/topic/not.20understanding.20deliberate.20error.20with.20.60ring.60.20over.20.E2.84.95/near/445879310) --- To make sure that the linter does not produce errors, #14007 activates the linter on "all" of mathlib. The expectation is that no error is thrown, just warnings. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-linter merge-conflict awaiting-author 251/0 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter/Papercut.lean,MathlibTest/Papercut.lean 4 24 ['Julian', 'YaelDillies', 'adomani', 'eric-wieser', 'github-actions'] nobody
83-70176
2 months ago
83-70176
2 months ago
7-47472
7 days
15991 vihdzp
author:vihdzp
feat(SetTheory/Ordinal/CantorNormalForm): alternate CNF recursion principle The idea of this recursion principle is that you can build an ordinal by adding one power of `b` at a time, as long as `1 < b ≤ ω`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-set-theory t-logic merge-conflict awaiting-author 43/0 Mathlib/SetTheory/Ordinal/Arithmetic.lean,Mathlib/SetTheory/Ordinal/CantorNormalForm.lean,Mathlib/SetTheory/Ordinal/Exponential.lean 3 8 ['YaelDillies', 'eric-wieser', 'github-actions', 'vihdzp'] nobody
83-31960
2 months ago
83-31960
2 months ago
91-50443
91 days
17758 vihdzp
author:vihdzp
feat(SetTheory/Ordinal/ENat): `Ordinal.toENat` We essentially copy the `Cardinal/ENat` file but make it for ordinals instead. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-set-theory merge-conflict 300/0 Mathlib.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/SetTheory/Cardinal/ENat.lean,Mathlib/SetTheory/Ordinal/Arithmetic.lean,Mathlib/SetTheory/Ordinal/Basic.lean,Mathlib/SetTheory/Ordinal/ENat.lean 6 2 ['Command-Master', 'github-actions', 'vihdzp'] nobody
83-31489
2 months ago
83-31489
2 months ago
126-40106
126 days
19698 vihdzp
author:vihdzp
refactor(SetTheory/Cardinal/Cofinality): redefine `Order.cof` We redefine `Order.cof` as a function on preorders, rather than one well-ordered relations. This allows us to use the `IsCofinal` API, alongside all the other goodies that come from a proper order structure. Finally, we clean up the `Ordinal.cof` API by relying on order results, rather than trying to haphazardly treat ordinals as sets. --- - [ ] depends on: #21972 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-set-theory merge-conflict WIP 502/583 Mathlib/Order/Cofinal.lean,Mathlib/SetTheory/Cardinal/Basic.lean,Mathlib/SetTheory/Cardinal/Cofinality.lean,Mathlib/SetTheory/Ordinal/Basic.lean 4 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
83-29500
2 months ago
83-29500
2 months ago
0-0
0 seconds
21856 vihdzp
author:vihdzp
chore(SetTheory/Cardinal/Basic): generalize universes of `sum_le_iSup_lift` We prove a more general version of the lemma which talks about families `ι → Cardinal.{v}` with `Small.{v} ι`, rather than just families `f : ι → Cardinal.{max u v}` with `ι : Type v`. We keep the old version, as it's seemingly more useful under common circumstances. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-set-theory merge-conflict 16/10 Mathlib/SetTheory/Cardinal/Basic.lean 1 6 ['b-mehta', 'github-actions', 'vihdzp'] nobody
83-29376
2 months ago
83-29376
2 months ago
32-26420
32 days
20967 joneugster
author:joneugster
tracking(CategoryTheory/Enriched/Limits): add conical limits Tracking PR for adding conical limits Co-authored-by: Emily Riehl Co-authored-by: Dagur Asgeirsson --- - [x] depends on: #20904 - [x] depends on: #20907 - [x] depends on: #20959 - [x] depends on: #20963 - [x] depends on: #20964 - [x] depends on: #20965 - content source: emilyriehl/infinity-cosmos#78 New implementation (not reflected on this branch yet): - [x] depends on: #22917 - [x] depends on: #22921 - [ ] depends on: #22923 - [ ] depends on: #22924 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) infinity-cosmos t-category-theory merge-conflict WIP 619/1 Mathlib.lean,Mathlib/CategoryTheory/Enriched/Limits/HasConicalLimits.lean,Mathlib/CategoryTheory/Enriched/Limits/HasConicalProducts.lean,Mathlib/CategoryTheory/Enriched/Limits/HasConicalPullbacks.lean,Mathlib/CategoryTheory/Enriched/Limits/HasConicalTerminal.lean,Mathlib/CategoryTheory/Enriched/Limits/IsConicalLimit.lean,Mathlib/CategoryTheory/Enriched/Limits/IsConicalTerminal.lean,Mathlib/CategoryTheory/Enriched/Ordinary/Basic.lean 8 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
82-75782
2 months ago
82-75784
2 months ago
0-0
0 seconds
19013 quangvdao
author:quangvdao
feat(Algebra/BigOperators/Fin): Add `finSigmaFinEquiv` This PR adds `finSigmaFinEquiv` which is the equivalence `(i : Fin m) × Fin (n i) ≃ Fin (∑ i, n i)`. This is the dependent version of `finProdFinEquiv`. CI should be passing, but there are two things I'd like feedback on: 1. When defining the mappings, I have to consider `m = 0` separately. Is there a more uniform definition? 2. I'm proving this as a step toward defining `Fin.join`, which is the analogue of `List.join`. I can now technically define `Fin.join` as: ``` variable {a : Fin n → ℕ} {α : (i : Fin n) → (j : Fin (a i)) → Sort*} def join (v : (i : Fin n) → (j : Fin (a i)) → α i j) (k : Fin (∑ i, a i)) : α (finSigmaFinEquiv.invFun k).1 (finSigmaFinEquiv.invFun k).2 := v (finSigmaFinEquiv.invFun k).1 (finSigmaFinEquiv.invFun k).2 ``` but this looks horrible. This highly motivates refactoring `invFun` as two new definitions: ``` def func1 {n : ℕ} (a : Fin n → ℕ) (k : Fin (∑ i, a i)) : Fin n := sorry def func2 {n : ℕ} (a : Fin n → ℕ) (k : Fin (∑ i, a i)) : Fin (a (func1 a k)) := sorry ``` I'm not sure what to call these functions. The analogues in the non-dependent case are `divNat` and `modNat`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict awaiting-author
label:t-algebra$
92/16 Mathlib/Algebra/BigOperators/Fin.lean 1 14 ['YaelDillies', 'eric-wieser', 'github-actions', 'quangvdao'] nobody
82-5809
2 months ago
82-5809
2 months ago
3-28829
3 days
20410 vihdzp
author:vihdzp
refactor: redefine `Equiv.Set.sumCompl = Equiv.sumCompl` It's still useful to have `Equiv.Set.sumCompl` around, as `simp` can't otherwise see through the def-eq `{x // x ∈ s} ⊕ {x // ¬ x ∈ s} = s ⊕ sᶜ`. --- - [ ] depends on: #20850 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data awaiting-CI merge-conflict blocked-by-other-PR WIP 33/21 Mathlib/Logic/Equiv/Basic.lean,Mathlib/Logic/Equiv/Fintype.lean,Mathlib/Logic/Equiv/Set.lean 3 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
81-53622
2 months ago
81-53622
2 months ago
0-0
0 seconds
20850 vihdzp
author:vihdzp
chore(Logic/Equiv/Basic): extend `sumCompl` API We make a couple of redundant arguments implicit, rename two misnamed theorems, and add two new ones. --- I'm not sure if the theorems I renamed actually had the correct name; if they did, then [`Equiv.Set.sumCompl_symm_apply_of_mem`](https://leanprover-community.github.io/mathlib4_docs/Mathlib/Logic/Equiv/Set.html#Equiv.Set.sumCompl_symm_apply_of_mem) and [`Equiv.Set.sumCompl_symm_apply_of_not_mem`](https://leanprover-community.github.io/mathlib4_docs/Mathlib/Logic/Equiv/Set.html#Equiv.Set.sumCompl_symm_apply_of_not_mem) should be renamed instead to match. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data t-logic merge-conflict awaiting-author 21/6 Mathlib/Logic/Equiv/Basic.lean,Mathlib/Logic/Equiv/Fintype.lean 2 5 ['eric-wieser', 'github-actions', 'grunweg', 'kbuzzard', 'vihdzp'] nobody
81-53498
2 months ago
81-53498
2 months ago
28-73677
28 days
20389 eric-wieser
author:eric-wieser
feat: generalize results to `WithLp 0` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis merge-conflict 116/53 Mathlib/Analysis/Normed/Lp/PiLp.lean 1 1 ['github-actions'] nobody
80-80757
2 months ago
80-80757
2 months ago
0-0
0 seconds
15915 vihdzp
author:vihdzp
chore(SetTheory/Ordinal/CantorNormalForm): `CNF.exponents` and `CNF.coeffs` We rewrite theorems about the Cantor Normal Form in terms of their lists of exponents and coefficients, instead of awkwardly talking about their first and second entries. We also put all theorems about the CNF in its own namespace. This keeps us from cluttering the `Ordinal` namespace, and it also avoids having to prefix everything by `CNF_` constantly. --- - [x] depends on: #16998 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-set-theory t-logic merge-conflict awaiting-author 117/44 Mathlib/SetTheory/Ordinal/CantorNormalForm.lean 1 32 ['Command-Master', 'YaelDillies', 'YnirPaz', 'digama0', 'github-actions', 'mathlib4-dependent-issues-bot', 'vihdzp'] nobody
80-62087
2 months ago
80-62087
2 months ago
53-79724
53 days
19189 YnirPaz
author:YnirPaz
feat(SetTheory/Ordinal/Arithmetic): order isomorphism between omega and the natural numbers --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-set-theory merge-conflict awaiting-author 44/0 Mathlib/Order/SuccPred/Limit.lean,Mathlib/SetTheory/Ordinal/Arithmetic.lean 2 21 ['YaelDillies', 'YnirPaz', 'github-actions', 'vihdzp'] nobody
80-61842
2 months ago
80-61842
2 months ago
47-37012
47 days
23145 joneugster
author:joneugster
feat(CategoryTheory/Enriched/Limits): add IsConicalLimits --- - [ ] depends on: #23142 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) infinity-cosmos t-category-theory merge-conflict blocked-by-other-PR 221/9 Mathlib.lean,Mathlib/CategoryTheory/Enriched/Limits/HasConicalLimits.lean,Mathlib/CategoryTheory/Enriched/Limits/IsConicalLimit.lean 3 3 ['github-actions', 'joelriou', 'mathlib4-dependent-issues-bot'] nobody
80-6600
2 months ago
80-6600
2 months ago
0-806
13 minutes
19227 adomani
author:adomani
fix(CI): unwrap `lake test` in problem matcher ... and also add a `#guard_msgs` in `AssertImported` test, so that `lake test` properly fails. [Zulip discussion](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/CI.3A.20noisy.20.22test.20mathlib.22/near/483126955) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) CI merge-conflict awaiting-author 9/20 .github/build.in.yml,.github/workflows/bors.yml,.github/workflows/build.yml,.github/workflows/build_fork.yml,MathlibTest/AssertImported.lean 5 2 ['bryangingechen', 'github-actions'] nobody
79-24845
2 months ago
79-24846
2 months ago
22-71271
22 days
20874 grunweg
author:grunweg
chore(nolint.yml): use shallow clones This should be sufficient, and be slightly faster on CI. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) CI merge-conflict awaiting-author 0/3 .github/workflows/nolints.yml 1 2 ['bryangingechen', 'github-actions'] nobody
79-24600
2 months ago
79-24600
2 months ago
0-15573
4 hours
21463 riccardobrasca
author:riccardobrasca
add algEquiv_comp_algebraMap --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-algebra t-number-theory merge-conflict WIP
label:t-algebra$
233/54 Mathlib.lean,Mathlib/RingTheory/DedekindDomain/IntegralClosure.lean,Mathlib/RingTheory/Ideal/Norm/RelNorm.lean,Mathlib/RingTheory/Localization/AtPrime.lean,Mathlib/RingTheory/Localization/Basic.lean,Mathlib/RingTheory/Localization/FractionRing.lean,Mathlib/RingTheory/Localization/LocalizationLocalization.lean,Mathlib/RingTheory/Localization/Separable.lean,Mathlib/RingTheory/RingHom/Finite.lean 9 4 ['github-actions', 'leanprover-bot', 'riccardobrasca'] nobody
77-11875
2 months ago
77-11875
2 months ago
0-1459
24 minutes
12664 BoltonBailey
author:BoltonBailey
feat: add lemma about `degreeOf_eq_degree` Adds `MvPolynomial.degreeOf_eq_degree`, which states that the degree of a particular variable in a multivariate polynomial is equal to the degree of the single-variable polynomial obtained by treating the multivariable polynomial as a single variable polynomial over multivariable polynomials in the remaining variables. needed by #11106 --- - [ ] depends on: #13861 [So that we can prove `optionEquivLeft_support` analogously to `finSuccEquiv_support`] [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict blocked-by-other-PR WIP
label:t-algebra$
50/0 Mathlib/Algebra/MvPolynomial/Equiv.lean 1 2 ['github-actions', 'leanprover-community-mathlib4-bot'] nobody
76-27451
2 months ago
91-7907
2 months ago
0-0
0 seconds
15774 kkytola
author:kkytola
feat: Topology on `ENat` This PR may contain some results that are not in the PR that adds a toppology on `ENat`. --- The immediate motivation is to be able to make the right continuity statement of the extended floor function on `ENNReal`, when this floor function is made `ENat`valued as suggested in the PR review of #15269. The API here is modelled on the early parts of [the corresponding ENNReal file](https://leanprover-community.github.io/mathlib4_docs/Mathlib/Topology/Instances/ENNReal.html#top), although much of this case is more trivial. - [x] depends on: #15380 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order t-topology merge-conflict WIP 161/9 Mathlib/Data/ENat/Basic.lean,Mathlib/Topology/Instances/ENat.lean 2 4 ['YaelDillies', 'github-actions', 'leanprover-community-mathlib4-bot'] nobody
74-68777
2 months ago
74-68777
2 months ago
0-6819
1 hour
18284 chrisflav
author:chrisflav
feat(AlgebraicGeometry): relative gluing of schemes We show https://stacks.math.columbia.edu/tag/01LH using #14208. This shall be used to construct the relative spectrum of a quasi-coherent algebra. --- - [ ] depends on: #14208 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebraic-geometry merge-conflict WIP 1393/7 Mathlib.lean,Mathlib/AlgebraicGeometry/Gluing.lean,Mathlib/AlgebraicGeometry/OpenImmersion.lean,Mathlib/AlgebraicGeometry/RelativeGluing.lean,Mathlib/AlgebraicGeometry/Sites/Representability.lean,Mathlib/CategoryTheory/Functor/FullyFaithful.lean,Mathlib/CategoryTheory/Limits/Shapes/Types.lean,Mathlib/CategoryTheory/MorphismProperty/Representable.lean 8 n/a ['github-actions', 'joelriou', 'mathlib4-dependent-issues-bot'] nobody
74-5129
2 months ago
unknown
unknown
16810 urkud
author:urkud
feat: define `(a : ENat) ^ (b : ENat)` The definition agrees with `Cardinal.toENat`, i.e., `#(α → β) = #β ^ #α`, where `#` is the not-yet-defined `ENat.card α = Cardinal.toENat (Cardinal.mk α)`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-set-theory t-data merge-conflict 51/0 Mathlib.lean,Mathlib/Data/ENat/Pow.lean 2 1 ['github-actions'] nobody
73-47970
2 months ago
73-47970
2 months ago
0-0
0 seconds
16009 Command-Master
author:Command-Master
acyclic graph --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-combinatorics merge-conflict WIP 232/0 Mathlib/Combinatorics/SimpleGraph/Acyclic.lean 1 1 ['github-actions'] nobody
73-16926
2 months ago
73-16926
2 months ago
0-0
0 seconds
22930 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. --- - [ ] depends on: #22931 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-algebra merge-conflict blocked-by-other-PR
label:t-algebra$
267/200 Mathlib/RingTheory/FinitePresentation.lean,Mathlib/RingTheory/FiniteType.lean,Mathlib/RingTheory/LocalProperties/Basic.lean,Mathlib/RingTheory/Localization/BaseChange.lean,Mathlib/RingTheory/RingHom/Finite.lean,Mathlib/RingTheory/RingHom/FinitePresentation.lean,Mathlib/RingTheory/RingHom/FiniteType.lean,Mathlib/RingTheory/TensorProduct/Basic.lean 8 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
70-76416
2 months ago
70-76416
2 months ago
0-1344
22 minutes
20613 grunweg
author:grunweg
chore: golf using `List.toArrayMap` --- Depends on batteries#1090 landing in mathlib. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import merge-conflict 27/21 Cache/Main.lean,Cache/Requests.lean,Mathlib/Lean/Meta/RefinedDiscrTree/Lookup.lean,Mathlib/Tactic/DeriveTraversable.lean,Mathlib/Tactic/Linter/TextBased.lean,Mathlib/Tactic/MoveAdd.lean,Mathlib/Tactic/ToAdditive/Frontend.lean,Mathlib/Util/CompileInductive.lean,Mathlib/Util/GetAllModules.lean,Mathlib/Util/Notation3.lean,scripts/autolabel.lean 11 2 ['github-actions', 'vihdzp'] nobody
70-67743
2 months ago
70-67743
2 months ago
22-82622
22 days
20222 eric-wieser
author:eric-wieser
feat: generalize lemmas about derivatives Rather than creating a huge diff by shuffling things around, this generalizes everything in-place and swaps between `section`s for topological and normed vector spaces. The rationale for this approach is that: * we may further generalize the results of this file, and this avoids us jumbling up the order multiple times unnecessarily. * this greatly reduces the chance of merge conflicts --- - [ ] depends on: #21065 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis merge-conflict blocked-by-other-PR 554/50 Mathlib/Analysis/Calculus/Deriv/Basic.lean,Mathlib/Analysis/Calculus/FDeriv/Basic.lean,MathlibTest/Recall.lean 3 8 ['adomani', 'eric-wieser', 'github-actions', 'leanprover-bot', 'mathlib4-dependent-issues-bot'] nobody
70-39045
2 months ago
70-39045
2 months ago
16-16341
16 days
18444 jjdishere
author:jjdishere
feat(Topology/Algebra): Krasner's lemma This PR defines the class `IsKrasner K L` and `IsKrasnerNorm K L`. And proves that given a complete nontrivially normed/rank-one-valued field, every algebraic normed/valued fields extension L/K satisfies `IsKrasner K L`. However, as the uniqueness extension of norm of such a field is not merged into Mathlib yet, we put this as a condition in the theorem. --- - [x] depends on: #18142 - [x] depends on: #18698 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-analysis t-topology t-number-theory merge-conflict WIP
label:t-algebra$
440/0 Mathlib.lean,Mathlib/Topology/Algebra/Krasner.lean 2 n/a ['github-actions', 'jjdishere', 'mathlib4-dependent-issues-bot'] nobody
70-25746
2 months ago
unknown
unknown
15989 vihdzp
author:vihdzp
feat(SetTheory/Ordinal/Principal): golf theorems on additively principal ordinals We add some new results on additively principal ordinals and use them to simplify existing theorems. --- - [x] depends on: #15990 - [x] depends on: #17740 - [x] depends on: #17741 - [x] depends on: #17742 - [x] depends on: #17842 - [x] depends on: #18902 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-set-theory t-logic merge-conflict awaiting-author 64/59 Mathlib/SetTheory/Ordinal/Arithmetic.lean,Mathlib/SetTheory/Ordinal/Notation.lean,Mathlib/SetTheory/Ordinal/Principal.lean 3 8 ['YaelDillies', 'github-actions', 'kbuzzard', 'mathlib4-dependent-issues-bot', 'vihdzp'] nobody
69-59586
2 months ago
69-59586
2 months ago
60-46576
60 days
22682 grunweg
author:grunweg
chore(Topology/Homeomorph): split out various constructions This makes `Homeomorph.lean` slightly more manageable, and also is a mild import reduction. edit: also split out IsHomeomorph, as this allows removing the dependencies on Constructions. Let's see if this gains much --- I don't feel strongly about this PR, but we might as well take it. - [ ] depends on: #22681 - [ ] depends on #22827 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) tech debt t-topology RFC merge-conflict 341/290 Mathlib.lean,Mathlib/Topology/Category/TopCat/ULift.lean,Mathlib/Topology/Homeomorph/Constructions.lean,Mathlib/Topology/Homeomorph/IsHomeomorph.lean,Mathlib/Topology/Homeomorph/Lemmas.lean,Mathlib/Topology/NoetherianSpace.lean 6 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
69-57349
2 months ago
69-57349
2 months ago
14-35834
14 days
21018 markimunro
author:markimunro
feat(Data/Matrix): add file with key definitions and theorems about elementary row operations Prove that each elementary row operation is equivalent to a multiplication by an elementary matrix, has another row operation which inverts it, and that each elementary matrix has a left inverse. This is a very large PR and I understand it will take time. This is my first one and will likely have issues but I will be ready to answer questions/fix them as soon as possible. Co-authored-by: Christopher Lynch --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data new-contributor merge-conflict awaiting-author enhancement 1230/0 Mathlib.lean,Mathlib/Data/Matrix/ElementaryRowOperations.lean,Mathlib/Data/Matrix/GaussianElimination.lean,Mathlib/Data/Matrix/GaussianEliminationOld,Mathlib/Data/Matrix/oldnames,et --hard 18533caba32,lean-toolchain 7 n/a ['chrisflav', 'eric-wieser', 'github-actions', 'j-loreaux', 'markimunro'] nobody
69-47112
2 months ago
unknown
unknown
23514 eric-wieser
author:eric-wieser
refactor: smooth over Lattice/LinearOrder inheritance This fixes the forgetful inheritance in `CompleteLinearOrder` and `ConditionallyCompleteLinearOrder`, which previously did not carry `compare` fields. (edit: moved to #23515) The following is the inheritance diagram before, where the dotted lines are manual instances. Note that every lattice typeclass that extends `LinearOrder` has to implement another dotted line edge, and remember to copy all the necessary data fields. ```mermaid graph TD LinearOrder --> Min,Max; LinearOrder --> PartialOrder; Lattice --> PartialOrder; CompleteLinearOrder --> Lattice; ConditionallyCompleteLinearOrder --> Lattice; LinearOrder-.-> Lattice; CompleteLinearOrder -.-> LinearOrder; ConditionallyCompleteLinearOrder -.-> LinearOrder; ``` This change introduces two new auxiliary typeclasses, to encapsulate these troublesome edges. `LinearOrderedLattice` can be thought of as `LinearOrder`, but with `sup`/`inf` instead of `min`/`max`. This is crucial, because it ensures the duplicate fields are merged in `extends CompleteLattice X, LinearOrderedLattice X`, which would not be the case for `extends CompleteLattice X, LinearOrder X`. The result is: ```mermaid graph TD LinearOrder --> Min,Max; LinearOrder --> LinearOrderBase; LinearOrderBase --> PartialOrder; Lattice --> PartialOrder; LinearOrderedLattice -.-> LinearOrder; LinearOrderedLattice --> LinearOrderBase; LinearOrderedLattice --> Lattice; CompleteLinearOrder --> LinearOrderedLattice; ConditionallyCompleteLinearOrder --> LinearOrderedLattice; ``` --- - [ ] depends on: #23515 - [ ] [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict 85/66 Mathlib/Algebra/Order/Group/Defs.lean,Mathlib/Algebra/Order/Monoid/Defs.lean,Mathlib/Order/Basic.lean,Mathlib/Order/CompleteLattice/Defs.lean,Mathlib/Order/ConditionallyCompleteLattice/Defs.lean,Mathlib/Order/Defs/LinearOrder.lean,Mathlib/Order/Lattice.lean 7 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
68-72942
2 months ago
68-72942
2 months ago
0-3019
50 minutes
19907 kim-em
author:kim-em
chore: remove some 'nonrec' `nonrec` is nearly always obfuscatory: it tells the reader "this apparent recursive call is not actually, but I'm going to leave you to guess what it is instead", when we could just disambiguate and tell the reader. However I'm not sure I have the patience to go through the remaining 600 uses. (A few are genuinely useful, but I guess less than 10%.) t-algebra merge-conflict
label:t-algebra$
38/38 Mathlib/Algebra/Category/ModuleCat/Differentials/Basic.lean,Mathlib/Algebra/Category/ModuleCat/Differentials/Presheaf.lean,Mathlib/Algebra/CharP/ExpChar.lean,Mathlib/Algebra/ContinuedFractions/Computation/Approximations.lean,Mathlib/Algebra/ContinuedFractions/ConvergentsEquiv.lean,Mathlib/Algebra/DualNumber.lean,Mathlib/Algebra/Quaternion.lean 7 2 ['github-actions', 'kim-em'] nobody
68-33315
2 months ago
68-33315
2 months ago
50-75559
50 days
20746 JLimperg
author:JLimperg
Aesop forward branch test --- This is not a real PR; I just want to benchmark this Aesop branch. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict 14/6 .github/workflows/build.yml,Mathlib/Data/Nat/Prime/Defs.lean,lake-manifest.json,lakefile.lean,scripts/bench/fake-root/lib/lean/libleanshared.so,scripts/bench/run 6 11 ['JLimperg', 'Kha', 'github-actions', 'leanprover-bot'] nobody
68-30348
2 months ago
126-13301
4 months ago
0-0
0 seconds
11768 JovanGerb
author:JovanGerb
feat: Interactive Library Rewrite This PR defines the `rw??` library rewrite tactic that uses my `RefinedDiscrTree`. This is a point&click tactic, letting the user click on subexpressions in the main goal. The results are sorted by relevance, and are separated into sections based on the matched pattern. It comes with a filter button that allows you to switch between the (default) filtered view, with removed duplicate lemmas and not showing lemma names, and the complete view. There is also a section for definitionally unfolding the selected expression - these rewrites do not correspond to a library lemma. --- - [ ] depends on: #11968 - [x] depends on: #12016 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-meta merge-conflict blocked-by-other-PR 2788/1253 Mathlib.lean,Mathlib/Lean/GoalsLocation.lean,Mathlib/Lean/Meta/RefinedDiscrTree.lean,Mathlib/Lean/Meta/RefinedDiscrTree/Basic.lean,Mathlib/Lean/Meta/RefinedDiscrTree/Encode.lean,Mathlib/Lean/Meta/RefinedDiscrTree/Initialize.lean,Mathlib/Lean/Meta/RefinedDiscrTree/Lookup.lean,Mathlib/Lean/Meta/RefinedDiscrTree/Pi.lean,Mathlib/Tactic.lean,Mathlib/Tactic/FunProp.lean,Mathlib/Tactic/FunProp/Elab.lean,Mathlib/Tactic/FunProp/StateList.lean,Mathlib/Tactic/FunProp/Theorems.lean,Mathlib/Tactic/FunProp/Types.lean,Mathlib/Tactic/Widget/InteractiveUnfold.lean,Mathlib/Tactic/Widget/LibraryRewrite.lean,Mathlib/Topology/Defs/Basic.lean,MathlibTest/LibraryRewrite.lean,MathlibTest/RefinedDiscrTree.lean,scripts/noshake.json 20 n/a ['JovanGerb', 'eric-wieser', 'fpvandoorn', 'github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot'] nobody
68-28146
2 months ago
unknown
unknown
22810 pechersky
author:pechersky
feat(Counterexamples): metric space not induced by norm Because the distance is not homogeneous --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) - [x] depends on: #22845 t-analysis t-topology merge-conflict WIP 202/1 Counterexamples.lean,Counterexamples/NotBoundedSMulMetricSpace.lean,Mathlib.lean,Mathlib/Analysis/Normed/PiNat.lean,Mathlib/Topology/Algebra/Module/LocallyConvex.lean,Mathlib/Topology/MetricSpace/Polish.lean 6 21 ['eric-wieser', 'github-actions', 'loefflerd', 'mathlib4-dependent-issues-bot', 'pechersky'] nobody
68-23004
2 months ago
68-23032
2 months ago
0-84180
23 hours
13124 FR-vdash-bot
author:FR-vdash-bot
chore: remove `CovariantClass` and `ContravariantClass` Lean cannot handle `CovariantClass` and `ContravariantClass` correctly - TC slowness - [Zulip](https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/TC.20slowness) - https://github.com/leanprover-community/mathlib4/issues/6646#issuecomment-1691792488 - It may also have made #6326 fail. - Needs a weird hack to find instance: #9252 --- - [x] depends on: #13154 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP 602/486 Mathlib/Algebra/AddConstMap/Basic.lean,Mathlib/Algebra/Algebra/Operations.lean,Mathlib/Algebra/Algebra/Subalgebra/Pointwise.lean,Mathlib/Algebra/BigOperators/Group/Finset/Basic.lean,Mathlib/Algebra/BigOperators/Group/Multiset/Basic.lean,Mathlib/Algebra/Group/Subgroup/Pointwise.lean,Mathlib/Algebra/Group/Submonoid/Pointwise.lean,Mathlib/Algebra/Group/UniqueProds/Basic.lean,Mathlib/Algebra/Module/Submodule/Pointwise.lean,Mathlib/Algebra/MonoidAlgebra/Degree.lean,Mathlib/Algebra/Order/AddTorsor.lean,Mathlib/Algebra/Order/Group/Action.lean,Mathlib/Algebra/Order/Group/DenselyOrdered.lean,Mathlib/Algebra/Order/Group/Units.lean,Mathlib/Algebra/Order/GroupWithZero/Canonical.lean,Mathlib/Algebra/Order/GroupWithZero/Unbundled.lean,Mathlib/Algebra/Order/GroupWithZero/WithZero.lean,Mathlib/Algebra/Order/Monoid/Defs.lean,Mathlib/Algebra/Order/Monoid/Unbundled/Basic.lean,Mathlib/Algebra/Order/Monoid/Unbundled/Defs.lean,Mathlib/Algebra/Order/Monoid/Unbundled/OrderDual.lean,Mathlib/Algebra/Order/Monoid/Unbundled/WithTop.lean,Mathlib/Algebra/Order/Ring/Defs.lean,Mathlib/Algebra/Order/Ring/WithTop.lean,Mathlib/Algebra/Ring/Subring/Pointwise.lean,Mathlib/Algebra/Ring/Subsemiring/Pointwise.lean,Mathlib/Analysis/SumOverResidueClass.lean,Mathlib/Data/DFinsupp/Lex.lean,Mathlib/Data/Finsupp/Lex.lean,Mathlib/Data/NNRat/Defs.lean,Mathlib/GroupTheory/OrderOfElement.lean,Mathlib/Order/Filter/IsBounded.lean,Mathlib/Order/Filter/Pointwise.lean,Mathlib/Probability/Kernel/Defs.lean,Mathlib/RingTheory/Ideal/Pointwise.lean,Mathlib/RingTheory/Valuation/ValuationSubring.lean,Mathlib/Topology/Algebra/Order/LiminfLimsup.lean 37 6 ['FR-vdash-bot', 'MichaelStollBayreuth', 'github-actions', 'leanprover-bot', 'mathlib4-dependent-issues-bot'] nobody
67-50981
2 months ago
67-50981
2 months ago
0-1769
29 minutes
20008 FLDutchmann
author:FLDutchmann
feat(NumberTheory): Selberg sieve This PR is a working draft of the full proof of the fundamental theorem of the Selberg sieve. I will create dependent PRs as I clean up the code. This work was used in the first proof of the prime number theorem in PNT+. --- - [x] depends on: #20025 - [x] depends on: #20026 - [x] depends on: #20779 - [x] depends on: #21880 - [ ] depends on: #22052 - [ ] depends on: #23635 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis t-number-theory merge-conflict awaiting-author blocked-by-other-PR 937/0 Mathlib/NumberTheory/SelbergSieve/Basic.lean,Mathlib/NumberTheory/SelbergSieve/Selberg.lean,docs/references.bib 3 3 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
67-14983
2 months ago
77-18908
2 months ago
0-0
0 seconds
23383 vlad902
author:vlad902
feat(GroupTheory): finitely generated groups are quotients of free groups on finite generators This is equivalent to the formulation that finitely generated groups/monoids are quotients of FreeGroups/Monoids over the same generators, though I think the phrasing as a surjective homomorphism is more useful. t-algebra merge-conflict
label:t-algebra$
29/0 Mathlib/GroupTheory/Finiteness.lean 1 1 ['github-actions'] nobody
67-1808
2 months ago
67-1808
2 months ago
0-0
0 seconds
20401 RemyDegenne
author:RemyDegenne
feat: add sigmaFinite_iUnion ```lean lemma sigmaFinite_iUnion (μ : Measure α) {s : ℕ → Set α} (h_meas : MeasurableSet (⋃ n, s n)) [∀ n, SigmaFinite (μ.restrict (s n))] : SigmaFinite (μ.restrict (⋃ n, s n)) ``` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-measure-probability merge-conflict awaiting-author 37/28 Mathlib/MeasureTheory/Decomposition/Exhaustion.lean,Mathlib/MeasureTheory/Measure/Typeclasses.lean 2 4 ['RemyDegenne', 'github-actions', 'sgouezel'] nobody
66-56135
2 months ago
66-56136
2 months ago
0-73190
20 hours
19275 eric-wieser
author:eric-wieser
fix: if nolint files change, do a full rebuild Otherwise CI will succeed when removing entries from the file, but fail later when someone changes something unrelated. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict delegated 8/0 lakefile.lean 1 20 ['YaelDillies', 'adomani', 'eric-wieser', 'github-actions', 'grunweg', 'mathlib-bors'] nobody
66-20303
2 months ago
66-20303
2 months ago
0-214
3 minutes
23499 riccardobrasca
author:riccardobrasca
feat: add `RingTheory.MvPowerSeries.rename` We add `RingTheory.MvPowerSeries.rename` copying the beginning of `RingTheory.MvPolynomial.rename`. --- This is just the beginning of the file, the point of the PR is to see if we want any design changes. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict WIP
label:t-algebra$
205/0 Mathlib.lean,Mathlib/RingTheory/MvPowerSeries/Basic.lean,Mathlib/RingTheory/MvPowerSeries/Evaluation.lean,Mathlib/RingTheory/MvPowerSeries/PiTopology.lean,Mathlib/RingTheory/MvPowerSeries/Rename.lean,Mathlib/RingTheory/MvPowerSeries/Substitution.lean 6 14 ['AntoineChambert-Loir', 'github-actions', 'riccardobrasca'] nobody
66-13166
2 months ago
66-13166
2 months ago
0-19825
5 hours
12251 ScottCarnahan
author:ScottCarnahan
refactor(RingTheory/HahnSeries) : several generalizations This PR is a container for several smaller PRs that refactor and generalize the existing Hahn series theory. It is (I think) all we need from Hahn series to get a palatable theory of vertex algebras off the ground (other prerequisites from Lie algebras will eventually come in a different PR). Major changes include: - equivalence between iterated Hahn series and Hahn series on Lex products. - introduce `orderTop` and `leadingCoeff` functions. Here, `orderTop` is a `WithTop Γ`-valued version of `order` that does not need `[Zero Γ]` and `leadingCoeff` returns the coefficient of the minimal element of support (or zero if empty). - introduce ordered and cancellative vector addition classes together with some basic theory e.g., finiteness of antidiagonals for partially well-ordered sets. - `HahnSeries Γ R`-module structure on `HahnModule Γ' R V`, when `Γ` is an `OrderedCancelAddCommMonoid`, `Γ'` is a `PartialOrder` with `OrderedCancelVAdd Γ Γ'`, `R` is a semiring, and `V` is an `R`-module. - Move `AddVal` to a separate file - the underlying function is just `orderTop`, but the description of the valuation needs an additional import and an `IsDomain` hypothesis. Results that depended on `AddVal` are changed to use `orderTop` and generalized. --- - [x] depends on: #10781 [HahnSeries on Lex product] - [x] depends on: #10846 [HahnModule] - [x] depends on: #11965 [orderTop] - [x] depends on: #11979 [OrderedVAdd] - [x] depends on: #12996 [leadingTerm] - [x] depends on: #16649 - [x] depends on: #16701 - [x] depends on: #17004 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order t-algebra merge-conflict WIP
label:t-algebra$
1059/97 Mathlib/RingTheory/HahnSeries/Addition.lean,Mathlib/RingTheory/HahnSeries/Basic.lean,Mathlib/RingTheory/HahnSeries/HEval.lean,Mathlib/RingTheory/HahnSeries/Multiplication.lean,Mathlib/RingTheory/HahnSeries/PowerSeries.lean,Mathlib/RingTheory/HahnSeries/Summable.lean 6 n/a ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
66-6724
2 months ago
unknown
unknown
21769 JovanGerb
author:JovanGerb
feat: extensible `push_neg` tactic This was started by point (3) of https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Possible.20improvements.20to.20Lean.2FMathlib/near/499085779 To be able to use `push_neg` more generally, this PR reimplements the tactic so that it is extensible. So, users can tag lemmas to be used by `push_neg`. This PR tags lemmas concerning empty/nonempty, subsingleton/nontrivial, and finite/infinite to be used in `push_neg`. Additionally, the tactic is extended to be able to push any constant that you want to push, and `push_neg` is now a macro for `push Not`. So far, I've tried to add lemmas for pushing `Real.log`. I could imagine it could also be used for `Real.exp`, `pow`, `mul`, `smul`, or even `Set.mem`. (the `Set.mem` lemmas are mostly tagged with `@[simp]` already, but `push_mem` could be more readable than `simp` or `dsimp`). Or a combination of pushing `Not` and `Set.compl` could be useful. The implementation is with the `simp` infrastructure, but instead of using post lemmas, like in `simp`, `push` uses `pre` lemmas, so we rewrite each expression before its subterms are rewritten. This is a more efficient way to "push" constants recursively. Most lemmas are added via the `@[push]` attribute, but a few cases require some special handling, so they are implemented "by hand" in a simproc that is tried after the `push` lemmas. For example the simproc simplifies `¬∀ n, p` ⇨ `∃ n, ¬p`, but, this is overridden by the `push` lemma that rewrites `¬(p → q)` ⇨ `p ∧ ¬q` (which doesn't apply at every forall) --- - [ ] depends on: #21965 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-meta merge-conflict blocked-by-other-PR 786/544 Archive/Imo/Imo1988Q6.lean,Archive/Imo/Imo2013Q5.lean,Archive/Imo/Imo2024Q3.lean,Archive/ZagierTwoSquares.lean,Counterexamples/Phillips.lean,Mathlib.lean,Mathlib/Algebra/BigOperators/Finprod.lean,Mathlib/Algebra/BigOperators/Group/Finset/Defs.lean,Mathlib/Algebra/CharP/MixedCharZero.lean,Mathlib/Algebra/Group/Action/Defs.lean,Mathlib/Algebra/Group/Basic.lean,Mathlib/Algebra/Group/Defs.lean,Mathlib/Algebra/Group/Pi/Basic.lean,Mathlib/Algebra/Group/Pointwise/Finset/Basic.lean,Mathlib/Algebra/GroupWithZero/Action/Defs.lean,Mathlib/Algebra/Lie/Submodule.lean,Mathlib/Algebra/Lie/Weights/Linear.lean,Mathlib/Algebra/Module/DedekindDomain.lean,Mathlib/Algebra/Order/Antidiag/Nat.lean,Mathlib/Algebra/Order/Archimedean/IndicatorCard.lean,Mathlib/Algebra/Order/GroupWithZero/Canonical.lean,Mathlib/Algebra/Order/Monoid/Canonical/Defs.lean,Mathlib/Algebra/Polynomial/Degree/Definitions.lean,Mathlib/Algebra/Ring/Commute.lean,Mathlib/Algebra/Ring/Defs.lean,Mathlib/AlgebraicTopology/DoldKan/Degeneracies.lean,Mathlib/Analysis/Analytic/OfScalars.lean,Mathlib/Analysis/Analytic/Order.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Order.lean,Mathlib/Analysis/Calculus/FDeriv/Norm.lean,Mathlib/Analysis/Complex/OpenMapping.lean,Mathlib/Analysis/Complex/Polynomial/UnitTrinomial.lean,Mathlib/Analysis/SpecialFunctions/Log/Basic.lean,Mathlib/Analysis/SpecialFunctions/MulExpNegMulSqIntegral.lean,Mathlib/Combinatorics/Enumerative/Composition.lean,Mathlib/Combinatorics/Enumerative/DyckWord.lean,Mathlib/Combinatorics/SimpleGraph/Acyclic.lean,Mathlib/Combinatorics/SimpleGraph/Diam.lean,Mathlib/Combinatorics/SimpleGraph/Path.lean,Mathlib/Combinatorics/SimpleGraph/Turan.lean,Mathlib/Computability/AkraBazzi/GrowsPolynomially.lean,Mathlib/Data/Analysis/Filter.lean,Mathlib/Data/ENat/Lattice.lean,Mathlib/Data/Finite/Defs.lean,Mathlib/Data/Finset/Card.lean,Mathlib/Data/Finset/Empty.lean,Mathlib/Data/Finset/Powerset.lean,Mathlib/Data/Finset/SDiff.lean,Mathlib/Data/Fintype/Basic.lean,Mathlib/Data/Fintype/Card.lean,Mathlib/Data/Fintype/Prod.lean,Mathlib/Data/Fintype/Sum.lean,Mathlib/Data/Nat/Defs.lean,Mathlib/Data/Nat/Factorization/PrimePow.lean,Mathlib/Data/Nat/Lattice.lean,Mathlib/Data/Nat/Order/Lemmas.lean,Mathlib/Data/Nat/PrimeFin.lean,Mathlib/Data/Ordmap/Ordset.lean,Mathlib/Data/Real/Archimedean.lean,Mathlib/Data/Set/Basic.lean,Mathlib/Data/Set/Insert.lean,Mathlib/Data/Set/Lattice.lean,Mathlib/Data/Set/Operations.lean,Mathlib/Data/ZMod/Basic.lean,Mathlib/Dynamics/OmegaLimit.lean,Mathlib/FieldTheory/JacobsonNoether.lean,Mathlib/Geometry/Manifold/ChartedSpace.lean,Mathlib/Geometry/Manifold/PartitionOfUnity.lean,Mathlib/GroupTheory/ArchimedeanDensely.lean,Mathlib/GroupTheory/OrderOfElement.lean,Mathlib/GroupTheory/Perm/ClosureSwap.lean,Mathlib/GroupTheory/SpecificGroups/Cyclic.lean,Mathlib/GroupTheory/SpecificGroups/ZGroup.lean,Mathlib/InformationTheory/Hamming.lean,Mathlib/LinearAlgebra/AffineSpace/AffineSubspace.lean,Mathlib/LinearAlgebra/Eigenspace/Zero.lean,Mathlib/LinearAlgebra/Matrix/SemiringInverse.lean,Mathlib/LinearAlgebra/Multilinear/Basic.lean,Mathlib/LinearAlgebra/Reflection.lean,Mathlib/Logic/IsEmpty.lean,Mathlib/Logic/Nontrivial/Defs.lean,Mathlib/MeasureTheory/Covering/Differentiation.lean,Mathlib/MeasureTheory/Decomposition/Lebesgue.lean,Mathlib/MeasureTheory/Function/ConvergenceInMeasure.lean,Mathlib/MeasureTheory/Function/UniformIntegrable.lean,Mathlib/MeasureTheory/Group/FundamentalDomain.lean,Mathlib/MeasureTheory/Integral/Bochner.lean,Mathlib/MeasureTheory/Integral/Lebesgue.lean,Mathlib/MeasureTheory/Measure/DiracProba.lean,Mathlib/MeasureTheory/Measure/Haar/NormedSpace.lean,Mathlib/MeasureTheory/Measure/MeasureSpace.lean,Mathlib/MeasureTheory/Measure/MeasureSpaceDef.lean,Mathlib/MeasureTheory/Measure/OpenPos.lean,Mathlib/MeasureTheory/Measure/Typeclasses.lean,Mathlib/MeasureTheory/OuterMeasure/Basic.lean,Mathlib/MeasureTheory/SetAlgebra.lean,Mathlib/ModelTheory/Ultraproducts.lean,Mathlib/NumberTheory/AbelSummation.lean,Mathlib/NumberTheory/ArithmeticFunction.lean,Mathlib/NumberTheory/Divisors.lean 149 4 ['adomani', 'github-actions', 'grunweg', 'mathlib4-dependent-issues-bot'] nobody
64-83010
2 months ago
64-83012
2 months ago
5-54179
5 days
22727 grunweg
author:grunweg
feat: rewrite the isolated by and colon linters in Lean --- - depends on #22726 - depends on: #22728 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-linter merge-conflict awaiting-author 128/96 Mathlib/AlgebraicTopology/SimplexCategory/GeneratorsRelations/Basic.lean,Mathlib/Data/Finsupp/AList.lean,Mathlib/Data/Int/ModEq.lean,Mathlib/Data/List/Nodup.lean,Mathlib/Data/List/TFAE.lean,Mathlib/Data/Matroid/Circuit.lean,Mathlib/Data/Matroid/Minor/Basic.lean,Mathlib/GroupTheory/Perm/Cycle/Factors.lean,Mathlib/LinearAlgebra/TensorProduct/Vanishing.lean,Mathlib/Order/KrullDimension.lean,Mathlib/Probability/Kernel/WithDensity.lean,Mathlib/RingTheory/NoetherNormalization.lean,Mathlib/Tactic/Linter/TextBased.lean,Mathlib/Topology/Sets/OpenCover.lean,scripts/lint-style.py 15 3 ['adomani', 'github-actions', 'grunweg'] nobody
64-82421
2 months ago
64-82421
2 months ago
10-50342
10 days
22027 vihdzp
author:vihdzp
chore(SetTheory/Ordinal/FixedPoint); review `Ordinal.nfp` API This PR does the following: - add `iff` variants of various theorems, renaming some in the process - weaken some assumptions slightly - golf throughout --- - [x] depends on: #22017 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-set-theory merge-conflict 64/61 Mathlib/Logic/Equiv/List.lean,Mathlib/SetTheory/Ordinal/FixedPoint.lean 2 3 ['github-actions', 'grunweg', 'mathlib4-dependent-issues-bot'] nobody
64-82294
2 months ago
67-49254
2 months ago
43-68322
43 days
15212 victorliu5296
author:victorliu5296
feat: Add fundamental theorem of calculus-2 for Banach spaces add the Mean Value Theorem for Banach spaces to the library and include reference for the theorem statement This theorem states that if `f : X → Y` is differentiable along the line segment from `a` to `b`, then the change in `f` equals the integral of its derivative along this path. This extends the mean value theorem to Banach spaces. This can be used for the eventual proof of the Newton-Kantorovich theorem with 1 constant contained inside the added reference. Here is the discussion on Zulipchat: https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/Contributing.20FTC-2.20for.20Banach.20spaces new-contributor t-measure-probability t-analysis merge-conflict awaiting-author 60/1 Mathlib/MeasureTheory/Integral/FundThmCalculus.lean 1 3 ['github-actions', 'hrmacbeth', 'victorliu5296'] nobody
64-42101
2 months ago
64-42101
2 months ago
51-85104
51 days
13861 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`. 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 do some light refactoring for succinctness, and put this any related preexisting lemmas in a new file to not trigger the linter. Needed by #12664 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data merge-conflict 204/62 Mathlib.lean,Mathlib/Algebra/Category/MonCat/Adjunctions.lean,Mathlib/Data/Finsupp/Basic.lean,Mathlib/Data/Finsupp/Option.lean,Mathlib/Data/Finsupp/Single.lean,Mathlib/LinearAlgebra/Finsupp/LinearCombination.lean 6 1 ['github-actions'] nobody
63-80879
2 months ago
63-80879
2 months ago
12-6613
12 days
21858 vihdzp
author:vihdzp
refactor(SetTheory/Ordinal/FixedPoint): redefine `Ordinal.deriv` We previously defined the [ordinal derivative](https://en.wikipedia.org/wiki/Normal_function#Properties) of a function as the unique normal function satisfying `deriv f 0 = nfp f 0` and `deriv f (o + 1) = nfp f (deriv f o)` (where `nfp f a` is the next fixed point of `f` that's `≥ a`). The motivation here was to give a "nice" junk value on non-normal functions (the function is normal no matter what). However, in practice, this definition makes it unwieldy to prove things, by either requiring a tedious zero/successor/limit argument, or requiring one to rewrite `deriv f = enumOrd (fixedPoints f)`. We can instead define `deriv f = enumOrd (fixedPoints f)`. At the cost of giving "worse" junk values (which we have no legitimate uses of), we're able to much more easily prove all the expected properties in the standard case where `f` is a normal function. Finally, we do some drive-by API cleanup. --- - [ ] depends on: #21860 - [ ] depends on: #21970 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-set-theory merge-conflict 216/262 Mathlib/Logic/Equiv/List.lean,Mathlib/SetTheory/Cardinal/Cofinality.lean,Mathlib/SetTheory/Ordinal/Enum.lean,Mathlib/SetTheory/Ordinal/FixedPoint.lean,Mathlib/SetTheory/Ordinal/Principal.lean,Mathlib/SetTheory/Ordinal/Veblen.lean 6 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
63-80341
2 months ago
63-80343
2 months ago
0-1601
26 minutes
22701 ctchou
author:ctchou
feat(Combinatorics): the Katona circle method This file formalizes the Katona circle method. From PlainCombi (LeanCamCombi): https://github.com/YaelDillies/LeanCamCombi/blob/master/LeanCamCombi/PlainCombi/KatonaCircle.lean Co-authored-by: Yaël Dillies new-contributor t-combinatorics merge-conflict 121/0 Mathlib.lean,Mathlib/Combinatorics/KatonaCircle.lean 2 1 ['github-actions'] nobody
63-78056
2 months ago
63-78056
2 months ago
30-8337
30 days
23402 mattrobball
author:mattrobball
refactor(LinearAlgebra.TensorProduct): make `TensorProduct` irreducible Mathematicians generally do not reason about tensor products using a particular model, precisely because the universal properties are more natural and the precise instantiations are too complicated for most purposes. Similarly, we shouldn't allow Lean to look inside `TensorProduct` and encourage building API on top of it to avoid definitional abuse. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict
label:t-algebra$
124/69 Mathlib/Algebra/Category/ModuleCat/ChangeOfRings.lean,Mathlib/Algebra/Category/ModuleCat/Monoidal/Basic.lean,Mathlib/Algebra/Category/Ring/Constructions.lean,Mathlib/LinearAlgebra/Alternating/DomCoprod.lean,Mathlib/LinearAlgebra/QuadraticForm/TensorProduct.lean,Mathlib/LinearAlgebra/QuadraticForm/TensorProduct/Isometries.lean,Mathlib/LinearAlgebra/TensorProduct/Basic.lean,Mathlib/LinearAlgebra/TensorProduct/Subalgebra.lean,Mathlib/LinearAlgebra/TensorProduct/Tower.lean,Mathlib/RingTheory/Bialgebra/TensorProduct.lean,Mathlib/RingTheory/Coalgebra/TensorProduct.lean,Mathlib/RingTheory/Kaehler/CotangentComplex.lean,Mathlib/RingTheory/Kaehler/JacobiZariski.lean,Mathlib/RingTheory/LocalRing/Module.lean,Mathlib/RingTheory/TensorProduct/Basic.lean 15 8 ['eric-wieser', 'github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'mattrobball'] nobody
63-46361
2 months ago
63-46362
2 months ago
0-0
0 seconds
23694 xroblot
author:xroblot
feat(NumberField/IsCM): compute the index of the subgroup of real units --- - [ ] depends on: #23674 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-number-theory merge-conflict blocked-by-other-PR 626/83 Mathlib/Algebra/Field/Equiv.lean,Mathlib/Algebra/Group/Invertible/Basic.lean,Mathlib/Algebra/Polynomial/Splits.lean,Mathlib/AlgebraicGeometry/Morphisms/Proper.lean,Mathlib/FieldTheory/Galois/Basic.lean,Mathlib/FieldTheory/LinearDisjoint.lean,Mathlib/FieldTheory/Normal/Basic.lean,Mathlib/GroupTheory/GroupAction/FixedPoints.lean,Mathlib/GroupTheory/Index.lean,Mathlib/GroupTheory/SpecificGroups/Cyclic.lean,Mathlib/LinearAlgebra/Dimension/Localization.lean,Mathlib/NumberTheory/NumberField/CMField.Lean,Mathlib/NumberTheory/NumberField/CanonicalEmbedding/FundamentalCone.lean,Mathlib/NumberTheory/NumberField/Embeddings.lean,Mathlib/NumberTheory/NumberField/Units/Basic.lean,Mathlib/RingTheory/Artinian/Ring.lean,Mathlib/RingTheory/IntegralClosure/Algebra/Defs.lean,Mathlib/RingTheory/IntegralClosure/IsIntegralClosure/Basic.lean,Mathlib/RingTheory/LinearDisjoint.lean,Mathlib/RingTheory/Localization/FractionRing.lean,Mathlib/RingTheory/Localization/Integral.lean,Mathlib/RingTheory/RootsOfUnity/Complex.lean,Mathlib/RingTheory/SimpleRing/Field.lean 23 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
63-30956
2 months ago
63-30959
2 months ago
0-637
10 minutes
23696 xroblot
author:xroblot
feat(NumberField/IsCM): compute ratio of regulators --- - [ ] depends on: #23694 - [ ] depends on: #23374 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-number-theory merge-conflict blocked-by-other-PR 1115/142 Mathlib/Algebra/Field/Equiv.lean,Mathlib/Algebra/Group/Invertible/Basic.lean,Mathlib/Algebra/Module/ZLattice/Basic.lean,Mathlib/Algebra/Module/ZLattice/Covolume.lean,Mathlib/Algebra/Polynomial/Splits.lean,Mathlib/AlgebraicGeometry/Morphisms/Proper.lean,Mathlib/FieldTheory/Galois/Basic.lean,Mathlib/FieldTheory/LinearDisjoint.lean,Mathlib/FieldTheory/Normal/Basic.lean,Mathlib/GroupTheory/GroupAction/FixedPoints.lean,Mathlib/GroupTheory/Index.lean,Mathlib/GroupTheory/SpecificGroups/Cyclic.lean,Mathlib/LinearAlgebra/Determinant.lean,Mathlib/LinearAlgebra/Dimension/Finite.lean,Mathlib/LinearAlgebra/Dimension/Localization.lean,Mathlib/LinearAlgebra/FreeModule/Finite/Quotient.lean,Mathlib/LinearAlgebra/Matrix/Determinant/Basic.lean,Mathlib/NumberTheory/NumberField/CMField.Lean,Mathlib/NumberTheory/NumberField/CanonicalEmbedding/FundamentalCone.lean,Mathlib/NumberTheory/NumberField/CanonicalEmbedding/NormLeOne.lean,Mathlib/NumberTheory/NumberField/Embeddings.lean,Mathlib/NumberTheory/NumberField/Units/Basic.lean,Mathlib/NumberTheory/NumberField/Units/DirichletTheorem.lean,Mathlib/NumberTheory/NumberField/Units/Regulator.lean,Mathlib/RingTheory/Artinian/Ring.lean,Mathlib/RingTheory/IntegralClosure/Algebra/Defs.lean,Mathlib/RingTheory/IntegralClosure/IsIntegralClosure/Basic.lean,Mathlib/RingTheory/LinearDisjoint.lean,Mathlib/RingTheory/Localization/FractionRing.lean,Mathlib/RingTheory/Localization/Integral.lean,Mathlib/RingTheory/RootsOfUnity/Complex.lean,Mathlib/RingTheory/SimpleRing/Field.lean,Mathlib/Topology/Homeomorph/Lemmas.lean 33 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
63-30956
2 months ago
63-30957
2 months ago
0-508
8 minutes
19695 Timeroot
author:Timeroot
feat(ModelTheory): Set.Definable is transitive Upstreamed from the [EquationalTheories](https://github.com/teorth/equational_theories) project. The main new theorem in this PR is `Set.Definable_trans`, which is that definability of sets in first order logic is transitive. The other work (in Syntax/Semantics) is pretty much all to facilitate that statement and proof. --- - [x] depends on: #19618 - [x] depends on: #23501 - [ ] depends on: #23502 - [ ] depends on: #23504 - [ ] depends on: #23506 large-import t-logic merge-conflict blocked-by-other-PR 557/6 Mathlib/Data/Rel.lean,Mathlib/ModelTheory/Definability.lean,Mathlib/ModelTheory/Semantics.lean,Mathlib/ModelTheory/Syntax.lean,scripts/noshake.json 5 36 ['Timeroot', 'awainverse', 'github-actions', 'madvorak', 'mathlib4-dependent-issues-bot'] nobody
63-18110
2 months ago
63-18112
2 months ago
34-66547
34 days
15943 urkud
author:urkud
feat: add `ProdQuotientMapSpace` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology merge-conflict 731/11 Mathlib.lean,Mathlib/Topology/Basic.lean,Mathlib/Topology/Compactness/Compact.lean,Mathlib/Topology/Maps/ProdQuotient.lean 4 2 ['github-actions', 'leanprover-community-bot-assistant'] nobody
62-60473
2 months ago
62-60476
2 months ago
0-0
0 seconds
23786 grunweg
author:grunweg
Mr librarynote def 2b --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import merge-conflict WIP 510/484 Archive/Imo/Imo2019Q2.lean,Mathlib/Algebra/Algebra/Basic.lean,Mathlib/Algebra/Algebra/Defs.lean,Mathlib/Algebra/Algebra/Equiv.lean,Mathlib/Algebra/Algebra/Hom.lean,Mathlib/Algebra/Algebra/NonUnitalHom.lean,Mathlib/Algebra/Algebra/NonUnitalSubalgebra.lean,Mathlib/Algebra/Algebra/ZMod.lean,Mathlib/Algebra/BigOperators/Group/Finset/Defs.lean,Mathlib/Algebra/Category/Ring/Limits.lean,Mathlib/Algebra/Colimit/Ring.lean,Mathlib/Algebra/EuclideanDomain/Basic.lean,Mathlib/Algebra/Field/MinimalAxioms.lean,Mathlib/Algebra/Field/Subfield/Defs.lean,Mathlib/Algebra/Group/Action/Defs.lean,Mathlib/Algebra/Group/Action/End.lean,Mathlib/Algebra/Group/Action/Hom.lean,Mathlib/Algebra/Group/Conj.lean,Mathlib/Algebra/Group/Defs.lean,Mathlib/Algebra/Group/Equiv/Defs.lean,Mathlib/Algebra/Group/Hom/Defs.lean,Mathlib/Algebra/Group/InjSurj.lean,Mathlib/Algebra/Group/MinimalAxioms.lean,Mathlib/Algebra/Group/Pointwise/Set/Basic.lean,Mathlib/Algebra/Group/Pointwise/Set/Scalar.lean,Mathlib/Algebra/Group/Submonoid/Operations.lean,Mathlib/Algebra/Group/Units/Defs.lean,Mathlib/Algebra/Group/Units/Hom.lean,Mathlib/Algebra/GroupWithZero/Action/Defs.lean,Mathlib/Algebra/GroupWithZero/Action/End.lean,Mathlib/Algebra/GroupWithZero/Basic.lean,Mathlib/Algebra/GroupWithZero/Defs.lean,Mathlib/Algebra/GroupWithZero/Equiv.lean,Mathlib/Algebra/GroupWithZero/InjSurj.lean,Mathlib/Algebra/GroupWithZero/Units/Basic.lean,Mathlib/Algebra/HierarchyDesign.lean,Mathlib/Algebra/Lie/Basic.lean,Mathlib/Algebra/Lie/Derivation/Basic.lean,Mathlib/Algebra/Lie/OfAssociative.lean,Mathlib/Algebra/Module/Defs.lean,Mathlib/Algebra/Module/Equiv/Defs.lean,Mathlib/Algebra/Module/NatInt.lean,Mathlib/Algebra/Module/Rat.lean,Mathlib/Algebra/Module/RingHom.lean,Mathlib/Algebra/Module/ZMod.lean,Mathlib/Algebra/NoZeroSMulDivisors/Basic.lean,Mathlib/Algebra/NoZeroSMulDivisors/Defs.lean,Mathlib/Algebra/Order/Field/Defs.lean,Mathlib/Algebra/Order/Group/Defs.lean,Mathlib/Algebra/Order/Group/InjSurj.lean,Mathlib/Algebra/Order/GroupWithZero/Canonical.lean,Mathlib/Algebra/Order/Hom/Basic.lean,Mathlib/Algebra/Order/Hom/Ring.lean,Mathlib/Algebra/Order/Kleene.lean,Mathlib/Algebra/Order/Module/Defs.lean,Mathlib/Algebra/Order/Monoid/Basic.lean,Mathlib/Algebra/Order/Monoid/Defs.lean,Mathlib/Algebra/Order/Monoid/Unbundled/ExistsOfLE.lean,Mathlib/Algebra/Order/Ring/Defs.lean,Mathlib/Algebra/Order/Ring/Star.lean,Mathlib/Algebra/Order/Star/Basic.lean,Mathlib/Algebra/Order/Sub/Basic.lean,Mathlib/Algebra/Ring/Action/Basic.lean,Mathlib/Algebra/Ring/Equiv.lean,Mathlib/Algebra/Ring/InjSurj.lean,Mathlib/Algebra/Ring/MinimalAxioms.lean,Mathlib/Algebra/Ring/Subring/Defs.lean,Mathlib/Algebra/Ring/Subsemiring/Defs.lean,Mathlib/Algebra/Star/NonUnitalSubalgebra.lean,Mathlib/Algebra/Star/StarAlgHom.lean,Mathlib/Algebra/Star/StarRingHom.lean,Mathlib/Algebra/Star/Subalgebra.lean,Mathlib/AlgebraicGeometry/Scheme.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Note.lean,Mathlib/Analysis/CStarAlgebra/Spectrum.lean,Mathlib/Analysis/Convex/Uniform.lean,Mathlib/Analysis/InnerProductSpace/Convex.lean,Mathlib/Analysis/InnerProductSpace/OfNorm.lean,Mathlib/Analysis/InnerProductSpace/Projection.lean,Mathlib/Analysis/Normed/Field/Basic.lean,Mathlib/Analysis/Normed/Group/Basic.lean,Mathlib/Analysis/Normed/Group/Constructions.lean,Mathlib/Analysis/Normed/Group/Seminorm.lean,Mathlib/Analysis/Normed/Group/Uniform.lean,Mathlib/Analysis/Normed/Lp/PiLp.lean,Mathlib/Analysis/Normed/Lp/ProdLp.lean,Mathlib/Analysis/Normed/Module/Basic.lean,Mathlib/Analysis/Normed/Operator/LinearIsometry.lean,Mathlib/Analysis/Normed/Order/Lattice.lean,Mathlib/Analysis/Normed/Ring/Basic.lean,Mathlib/Analysis/RCLike/Lemmas.lean,Mathlib/CategoryTheory/Category/Basic.lean,Mathlib/CategoryTheory/Comma/Over/OverClass.lean,Mathlib/CategoryTheory/Monoidal/Skeleton.lean,Mathlib/CategoryTheory/MorphismProperty/Comma.lean,Mathlib/Data/Fintype/Card.lean,Mathlib/Data/FunLike/Fintype.lean,Mathlib/Data/NNRat/Defs.lean,Mathlib/Data/Nat/Cast/Defs.lean,Mathlib/Data/Nat/Init.lean 180 2 ['github-actions', 'leanprover-community-bot-assistant'] nobody
62-52574
2 months ago
62-52576
2 months ago
0-0
0 seconds
23411 PatrickMassot
author:PatrickMassot
chore: remove finiteness from Order.Filter.Lift Co-authored-by: Anatole Dedecker --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) longest-pole t-topology merge-conflict 48/21 Mathlib/Dynamics/TopologicalEntropy/DynamicalEntourage.lean,Mathlib/Order/Filter/Basic.lean,Mathlib/Order/Filter/Finite.lean,Mathlib/Order/Filter/Lift.lean,Mathlib/Order/Filter/SmallSets.lean,Mathlib/Topology/Algebra/ContinuousMonoidHom.lean,Mathlib/Topology/Basic.lean 7 4 ['Vierkantor', 'github-actions', 'kim-em', 'leanprover-community-bot-assistant'] nobody
62-38370
2 months ago
62-57939
2 months ago
10-21608
10 days
23831 vasnesterov
author:vasnesterov
feat(Analysis): binomial series convergence Prove * `one_add_cpow_hasFPowerSeriesOnBall_zero`: for complex `a` and `|x| < 1`, the binomial series converges to `(1 + x).cpow a`. * `one_add_rpow_hasFPowerSeriesOnBall_zero`: the variant of the above for reals. --- - [ ] depends on: #22538 - [ ] depends on: #23749 - [ ] depends on: #23790 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis merge-conflict blocked-by-other-PR 606/6 Mathlib.lean,Mathlib/Analysis/Analytic/Basic.lean,Mathlib/Analysis/Analytic/Binomial.lean,Mathlib/Analysis/Analytic/ChangeOrigin.lean,Mathlib/Analysis/Analytic/Constructions.lean,Mathlib/Analysis/Calculus/FormalMultilinearSeries.lean,Mathlib/Analysis/Calculus/IteratedDeriv/Defs.lean,Mathlib/Analysis/Calculus/IteratedDeriv/Lemmas.lean,Mathlib/Analysis/NormedSpace/Connected.lean,Mathlib/NumberTheory/NumberField/CanonicalEmbedding/Basic.lean,Mathlib/RingTheory/Binomial.lean,scripts/noshake.json 12 2 ['leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
62-18755
2 months ago
62-18756
2 months ago
0-822
13 minutes
22579 kvanvels
author:kvanvels
doc(Topology/Defs/Induced): fix comments on three functions related to RestrictGenTopology --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology merge-conflict awaiting-author documentation 10/9 Mathlib/Topology/Defs/Induced.lean,Mathlib/Topology/RestrictGen.lean 2 4 ['github-actions', 'kvanvels', 'leanprover-community-bot-assistant', 'urkud'] nobody
61-49004
2 months ago
61-49006
2 months ago
12-18679
12 days
19771 robertylewis
author:robertylewis
perf: qqify two functions in linarith --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta merge-conflict 17/24 Mathlib/Tactic/Linarith/Frontend.lean,Mathlib/Tactic/Linarith/Verification.lean 2 5 ['github-actions', 'grunweg', 'leanprover-bot', 'leanprover-community-bot-assistant', 'robertylewis'] nobody
61-28510
2 months ago
61-28511
2 months ago
0-0
0 seconds
22308 plp127
author:plp127
feat (Analysis/Convex): Generalize `Convex` lemmas to `StarConvex` This PR generalizes many lemmas assuming `Convex 𝕜 s` to assume `StarConvex 𝕜 0 s`. --- - [x] depends on: #22421 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-analysis merge-conflict WIP 30/18 Mathlib/Analysis/Convex/Gauge.lean,Mathlib/Analysis/Convex/GaugeRescale.lean,Mathlib/Analysis/Convex/Star.lean,Mathlib/Analysis/LocallyConvex/AbsConvexOpen.lean 4 5 ['Paul-Lez', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
61-28021
2 months ago
61-28023
2 months ago
0-0
0 seconds
21488 imbrem
author:imbrem
feat(CategoryTheory/Monoidal): premonoidal categories Add support for premonoidal categories --- Still want to add support for: - Premonoidal braided/symmetric categories - The monoidal coherence theorem, which I've already ported in my `discretion` library - The `coherence` tactic, which should work fine for premonoidal categories too but wanted to get this in front of reviewers ASAP to make sure my general approach was alright [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-category-theory merge-conflict 900/361 Mathlib/Algebra/Category/ModuleCat/Presheaf/Monoidal.lean,Mathlib/CategoryTheory/Bicategory/End.lean,Mathlib/CategoryTheory/GradedObject/Monoidal.lean,Mathlib/CategoryTheory/Localization/Monoidal.lean,Mathlib/CategoryTheory/Monoidal/Braided/Basic.lean,Mathlib/CategoryTheory/Monoidal/Category.lean,Mathlib/CategoryTheory/Monoidal/Center.lean,Mathlib/CategoryTheory/Monoidal/CoherenceLemmas.lean,Mathlib/CategoryTheory/Monoidal/Discrete.lean,Mathlib/CategoryTheory/Monoidal/End.lean,Mathlib/CategoryTheory/Monoidal/Free/Basic.lean,Mathlib/CategoryTheory/Monoidal/Functor.lean,Mathlib/CategoryTheory/Monoidal/FunctorCategory.lean,Mathlib/CategoryTheory/Monoidal/Mon_.lean,Mathlib/CategoryTheory/Monoidal/Opposite.lean,Mathlib/CategoryTheory/Monoidal/Transport.lean,Mathlib/Tactic/CategoryTheory/Monoidal/Datatypes.lean,Mathlib/Tactic/CategoryTheory/Monoidal/Normalize.lean,Mathlib/Tactic/CategoryTheory/Monoidal/PureCoherence.lean,Mathlib/Tactic/CategoryTheory/MonoidalComp.lean,MathlibTest/StringDiagram.lean 21 9 ['YaelDillies', 'github-actions', 'grunweg', 'imbrem', 'kim-em', 'leanprover-community-bot-assistant'] nobody
61-24289
2 months ago
61-24290
2 months ago
58-20339
58 days
21525 sinhp
author:sinhp
feat(CategoryTheory): Locally Cartesian Closed Categories (Prelim) This PR defines the basic preliminaries for defining locally cartesian closed categories (LCCCs). In particular, using the calculus of mates we define certain natural isomorphisms involving `Over.star` and `Over.pullback` which will be crucial in defining the right adjoint to the pullback functor in the development of LCCCs. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-category-theory merge-conflict 338/24 Mathlib/CategoryTheory/Comma/Over/Basic.lean,Mathlib/CategoryTheory/Comma/Over/Pullback.lean,Mathlib/CategoryTheory/Galois/Examples.lean 3 13 ['b-mehta', 'github-actions', 'joelriou', 'leanprover-community-bot-assistant', 'sinhp'] nobody
61-24287
2 months ago
61-24289
2 months ago
43-83249
43 days
22319 sinhp
author:sinhp
feat(CategoryTheory): Locally Cartesian Closed Categories (Sections Right Adjoint) we define the `Over.sections` functor in the file `CategoryTheory.Comma.Over.Sections` and prove that it is a right adjoint to the `Over.star`, thereby solving an existing TODO in `Over.pullback` file. The `sections` functor is used to define the right adjoint to the pullback functor `Over.pullback` in the development of LCCCs. Moreover, the rest of added lemmas and theorems to `CategoryTheory.Comma.Over.Pullback` are crucial for the development of LCCCs in the next PR. --- - [ ] depends on: #21525 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-category-theory merge-conflict blocked-by-other-PR 547/24 Mathlib.lean,Mathlib/CategoryTheory/Comma/Over/Basic.lean,Mathlib/CategoryTheory/Comma/Over/Pullback.lean,Mathlib/CategoryTheory/Comma/Over/Sections.lean,Mathlib/CategoryTheory/Galois/Examples.lean 5 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
61-23760
2 months ago
61-23762
2 months ago
0-2084
34 minutes
22321 sinhp
author:sinhp
feat(CategoryTheory): Locally Cartesian Closed Categories (Definition) This PR defines locally cartesian closed categories in terms of existence of the pushforward functors (right adjoint to the pullback functor) for all morphisms. We develop basic API and prove the following: 1. Existence of the pushforward functors is equivalent to cartesian closed slices. 2. Any locally cartesian closed category with a terminal object is cartesian closed. 3. The slices of a locally cartesian closed category are locally cartesian closed. Some of the content is based on the project of formalization of polynomial functors at the Trimester "Prospect of Formal Mathematics" at the Hausdorff Institute (HIM) in Bonn. https://github.com/sinhp/Poly I found this implementation of locally cartesian closed categories amenable to polynomial functors formalization. Co-authored-by: Emily Riehl --- - [ ] depends on: #21525 - [ ] depends on: #22319 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-category-theory merge-conflict blocked-by-other-PR 812/24 Mathlib.lean,Mathlib/CategoryTheory/Comma/Over/Basic.lean,Mathlib/CategoryTheory/Comma/Over/Pullback.lean,Mathlib/CategoryTheory/Comma/Over/Sections.lean,Mathlib/CategoryTheory/Galois/Examples.lean,Mathlib/CategoryTheory/LocallyCartesianClosed/Basic.lean 6 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
61-23760
2 months ago
61-23761
2 months ago
0-336
5 minutes
13653 adomani
author:adomani
feat: the unusedSetOptionIn linter --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-linter merge-conflict 199/0 Mathlib.lean,Mathlib/Algebra/Homology/HomotopyCategory/Triangulated.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter.lean,Mathlib/Tactic/Linter/UnnecessarySetOptionIn.lean,MathlibTest/UnnecessarySetOptionIn.lean 6 15 ['adomani', 'github-actions', 'grunweg', 'leanprover-community-bot-assistant'] nobody
60-55125
1 month ago
60-55127
1 month ago
0-0
0 seconds
23374 xroblot
author:xroblot
feat(NumberField/Units): compute index of unit subgroups using regulators --- - [ ] depends on: #23312 - [ ] depends on: #22961 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-number-theory merge-conflict blocked-by-other-PR 413/59 Mathlib/Algebra/Module/ZLattice/Basic.lean,Mathlib/Algebra/Module/ZLattice/Covolume.lean,Mathlib/GroupTheory/Index.lean,Mathlib/LinearAlgebra/Determinant.lean,Mathlib/LinearAlgebra/Dimension/Finite.lean,Mathlib/LinearAlgebra/FreeModule/Finite/Quotient.lean,Mathlib/LinearAlgebra/Matrix/Determinant/Basic.lean,Mathlib/NumberTheory/NumberField/CanonicalEmbedding/NormLeOne.lean,Mathlib/NumberTheory/NumberField/Units/DirichletTheorem.lean,Mathlib/NumberTheory/NumberField/Units/Regulator.lean,Mathlib/Topology/Homeomorph/Lemmas.lean 11 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
60-51088
1 month ago
60-51090
1 month ago
0-177
2 minutes
19425 hrmacbeth
author:hrmacbeth
perf: gcongr forward-reasoning adjustment This PR changes the "forward-reasoning" component of `gcongr`, rendering it more efficient, particularly in problems with a large number of variables/hypotheses in the context. Previously `gcongr` attempted to match *every* `LocalDecl` against *every* node in the parse tree using *each* of the five implemented `@[gcongr_forward]` mini-tactics: matching directly, matching after applying `symm`, matching after applying `le_of_lt`, etc etc. The new algorithm filters out the non-Prop `LocalDecl`s, and also adjusts the `@[gcongr_forward]` extensions so that, rather than re-apply the relevant lemmas (`symm`, `le_of_lt`, etc) at every node in the parse tree, the lemmas are applied in advance to the `LocalDecl`s and the result (if successful) stored. The performance effect on mathlib as a whole is miniscule, but it speeds up the profiler's count of "tactic execution of Mathlib.Tactic.GCongr" in the newly-added test from 257 ms to 47 ms, and has a similar effect on real-life examples in an analysis project of mine. Co-authored-by: Mario Carneiro --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) (Note that Mario provided the ideas but not the code, so please review with appropriate diligence!) merge-conflict awaiting-author 130/59 Mathlib/Order/Lattice.lean,Mathlib/Tactic/GCongr/Core.lean,Mathlib/Tactic/GCongr/ForwardAttr.lean,MathlibTest/GCongr/inequalities.lean 4 17 ['Vierkantor', 'github-actions', 'hrmacbeth', 'leanprover-bot', 'leanprover-community-bot-assistant'] Vierkantor
assignee:Vierkantor
60-36821
1 month ago
60-36823
1 month ago
4-16654
4 days
20873 vbeffara
author:vbeffara
feat(Topology/Covering): path lifting and homotopy lifting This proves the existence and uniqueness of path and homotopy lifts through covering maps. --- I tried to separate as much of the proof as possible into separate PRs (which are already in Mathlib now), but the proof here relies on a monolithic construction of an explicit lift along a well-chosen subdivision, in `partial_lift`, with associated definitions. Only one standalone lean file added. An older WIP PR #10084 by Junyan Xu @alreadydone proves similar results using a very similar construction for path lifting, with a different argument to obtain continuity for homotopy lifting. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-topology merge-conflict awaiting-author 281/1 Mathlib.lean,Mathlib/Topology/Covering/Basic.lean,Mathlib/Topology/Covering/Lift.lean 3 9 ['alreadydone', 'github-actions', 'grunweg', 'vbeffara'] nobody
60-27017
1 month ago
60-27017
1 month ago
55-53553
55 days
22817 peabrainiac
author:peabrainiac
feat(CategoryTheory/Sites): local sites Defines local sites and shows that sheaves of types on them form a local topos, in that the global sections functor `Sheaf.Γ` has a right adjoint `Sheaf.codisc` that is fully faithful. --- - [x] depends on: #22816 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory merge-conflict WIP 263/0 Mathlib.lean,Mathlib/CategoryTheory/Limits/FunctorCategory/Shapes/Products.lean,Mathlib/CategoryTheory/Limits/Types.lean,Mathlib/CategoryTheory/Sites/GlobalSections.lean,Mathlib/CategoryTheory/Sites/LocalSite.lean,Mathlib/CategoryTheory/Sites/Sheaf.lean 6 4 ['github-actions', 'joelriou', 'mathlib4-dependent-issues-bot'] nobody
59-47026
1 month ago
59-50549
1 month ago
0-568
9 minutes
6252 michaellee94
author:michaellee94
feat(Geometry/Manifolds/Instances/Homeomorph): Homeomorphism maps `C^k` manifolds to `C^k` manifolds --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-differential-geometry merge-conflict WIP 116/0 Mathlib.lean,Mathlib/Geometry/Manifold/Instances/Graph.lean 2 2 ['leanprover-community-bot-assistant', 'michaellee94'] nobody
59-21482
1 month ago
59-21484
1 month ago
1-44375
1 day
22059 grunweg
author:grunweg
feat: manifolds with smooth boundary Needs polish, and closing the remaining sorries (or deciding they can be postponed later). From my bordism theory project. --- - [x] depends on: #22070 - [x] depends on: #22128 - [x] depends on: #22131 - [x] depends on: #22082 - [x] depends on: #22113 - [x] depends on: #22105 - [ ] depends on: #22137 - [ ] depends on: #22642 (and a similar result for direct sums), still WIP - [ ] depends on #23040 for the mathlib-level definition of smooth immersions and embeddings [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-differential-geometry merge-conflict blocked-by-other-PR WIP 603/0 Mathlib.lean,Mathlib/Geometry/Manifold/HasSmoothBoundary.lean 2 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
59-19736
1 month ago
59-19738
1 month ago
0-0
0 seconds
7873 FR-vdash-bot
author:FR-vdash-bot
perf: reorder `extends` and change instance priority in algebra hierarchy There are no strict rules, but in general `Cancel` is dropped first, then `Comm`, then `Neg / Inv`, then `Assoc`. Not sure if there's a better way. --- - [ ] depends on: #14712 - [x] depends on: #16638 - [ ] depends on: #18464 - [ ] depends on: #18468 - [ ] depends on: #18470 - [ ] depends on: #18472 - [ ] depends on: #18474 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) slow-typeclass-synthesis t-algebra merge-conflict blocked-by-other-PR
label:t-algebra$
494/204 Archive/Imo/Imo1998Q2.lean,Mathlib/Algebra/Algebra/Hom.lean,Mathlib/Algebra/Associated.lean,Mathlib/Algebra/BigOperators/Ring/List.lean,Mathlib/Algebra/Category/ModuleCat/Presheaf/Limits.lean,Mathlib/Algebra/DirectSum/Algebra.lean,Mathlib/Algebra/DirectSum/Internal.lean,Mathlib/Algebra/EuclideanDomain/Defs.lean,Mathlib/Algebra/EuclideanDomain/Field.lean,Mathlib/Algebra/Field/Basic.lean,Mathlib/Algebra/Field/Defs.lean,Mathlib/Algebra/Field/IsField.lean,Mathlib/Algebra/GCDMonoid/Basic.lean,Mathlib/Algebra/Group/Defs.lean,Mathlib/Algebra/Group/Ext.lean,Mathlib/Algebra/Group/InjSurj.lean,Mathlib/Algebra/Group/Opposite.lean,Mathlib/Algebra/Group/Prod.lean,Mathlib/Algebra/GroupWithZero/Basic.lean,Mathlib/Algebra/GroupWithZero/Defs.lean,Mathlib/Algebra/GroupWithZero/InjSurj.lean,Mathlib/Algebra/GroupWithZero/Prod.lean,Mathlib/Algebra/GroupWithZero/Semiconj.lean,Mathlib/Algebra/GroupWithZero/Units/Basic.lean,Mathlib/Algebra/Homology/Embedding/Basic.lean,Mathlib/Algebra/Homology/HomotopyCategory/DegreewiseSplit.lean,Mathlib/Algebra/Homology/HomotopyCategory/ShiftSequence.lean,Mathlib/Algebra/Lie/Basic.lean,Mathlib/Algebra/MonoidAlgebra/Grading.lean,Mathlib/Algebra/Order/AddGroupWithTop.lean,Mathlib/Algebra/Order/Field/Canonical/Defs.lean,Mathlib/Algebra/Order/Field/Defs.lean,Mathlib/Algebra/Order/Group/Abs.lean,Mathlib/Algebra/Order/Group/Defs.lean,Mathlib/Algebra/Order/GroupWithZero/Canonical.lean,Mathlib/Algebra/Order/Kleene.lean,Mathlib/Algebra/Order/Monoid/Defs.lean,Mathlib/Algebra/Order/Ring/Canonical.lean,Mathlib/Algebra/Order/Ring/Defs.lean,Mathlib/Algebra/Polynomial/Roots.lean,Mathlib/Algebra/Quaternion.lean,Mathlib/Algebra/Ring/BooleanRing.lean,Mathlib/Algebra/Ring/Defs.lean,Mathlib/Algebra/Ring/Ext.lean,Mathlib/Algebra/Ring/InjSurj.lean,Mathlib/Algebra/Ring/Rat.lean,Mathlib/Algebra/Tropical/Basic.lean,Mathlib/Analysis/Fourier/FourierTransformDeriv.lean,Mathlib/Analysis/InnerProductSpace/Orientation.lean,Mathlib/Analysis/InnerProductSpace/Symmetric.lean,Mathlib/Analysis/Normed/Field/Basic.lean,Mathlib/Analysis/Normed/Group/Basic.lean,Mathlib/Analysis/NormedSpace/Star/Multiplier.lean,Mathlib/CategoryTheory/Preadditive/FunctorCategory.lean,Mathlib/CategoryTheory/Preadditive/SingleObj.lean,Mathlib/CategoryTheory/Triangulated/Functor.lean,Mathlib/Data/Finset/NoncommProd.lean,Mathlib/Data/Int/Cast/Defs.lean,Mathlib/Data/Nat/Cast/Defs.lean,Mathlib/Data/Nat/Choose/Multinomial.lean,Mathlib/Data/Num/Lemmas.lean,Mathlib/Data/Rat/Denumerable.lean,Mathlib/Data/Real/ENatENNReal.lean,Mathlib/Dynamics/Ergodic/AddCircle.lean,Mathlib/FieldTheory/KummerExtension.lean,Mathlib/GroupTheory/Congruence/Basic.lean,Mathlib/GroupTheory/MonoidLocalization.lean,Mathlib/GroupTheory/SpecificGroups/Alternating.lean,Mathlib/GroupTheory/Torsion.lean,Mathlib/Init/ZeroOne.lean,Mathlib/LinearAlgebra/LinearPMap.lean,Mathlib/LinearAlgebra/Orientation.lean,Mathlib/LinearAlgebra/QuadraticForm/Basic.lean,Mathlib/LinearAlgebra/TensorPower.lean,Mathlib/LinearAlgebra/TensorProduct/Basic.lean,Mathlib/LinearAlgebra/TensorProduct/Graded/External.lean,Mathlib/MeasureTheory/Decomposition/Jordan.lean,Mathlib/MeasureTheory/Decomposition/SignedLebesgue.lean,Mathlib/NumberTheory/ArithmeticFunction.lean,Mathlib/NumberTheory/LegendreSymbol/GaussEisensteinLemmas.lean,Mathlib/NumberTheory/RamificationInertia.lean,Mathlib/NumberTheory/WellApproximable.lean,Mathlib/NumberTheory/Zsqrtd/QuadraticReciprocity.lean,Mathlib/Order/Filter/Germ.lean,Mathlib/Order/Interval/Finset/Box.lean,Mathlib/RingTheory/Bialgebra/Hom.lean,Mathlib/RingTheory/Coalgebra/Hom.lean,Mathlib/RingTheory/DiscreteValuationRing/Basic.lean,Mathlib/RingTheory/Filtration.lean,Mathlib/RingTheory/Henselian.lean,Mathlib/RingTheory/Ideal/IsPrincipal.lean,Mathlib/RingTheory/Ideal/LocalRing.lean,Mathlib/RingTheory/Ideal/Norm.lean,Mathlib/RingTheory/Localization/Integral.lean,Mathlib/RingTheory/MvPolynomial/Symmetric.lean,Mathlib/RingTheory/TensorProduct/Basic.lean,Mathlib/RingTheory/TensorProduct/MvPolynomial.lean,Mathlib/RingTheory/UniqueFactorizationDomain.lean,Mathlib/RingTheory/Valuation/ValuationSubring.lean,Mathlib/Tactic/Positivity/Core.lean 104 84 ['FR-vdash-bot', 'MichaelStollBayreuth', 'github-actions', 'kim-em', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'mattrobball'] nobody
59-858
1 month ago
328-69191
10 months ago
7-77799
7 days
23867 kim-em
author:kim-em
chore: remove unnecessary `[AtLeastTwo n]` hypotheses This PR is a follow-up to #23866, demonstrating that we can remove nearly all the `[AtLeastTwo n]` hypotheses across Mathlib. bench-after-CI merge-conflict 272/278 Mathlib/Algebra/AddConstMap/Basic.lean,Mathlib/Algebra/CharP/Defs.lean,Mathlib/Algebra/CharP/Invertible.lean,Mathlib/Algebra/DirectSum/Internal.lean,Mathlib/Algebra/DirectSum/Ring.lean,Mathlib/Algebra/Group/Hom/End.lean,Mathlib/Algebra/Group/Opposite.lean,Mathlib/Algebra/Group/ULift.lean,Mathlib/Algebra/Module/LinearMap/End.lean,Mathlib/Algebra/Module/NatInt.lean,Mathlib/Algebra/MonoidAlgebra/ToDirectSum.lean,Mathlib/Algebra/Order/Floor/Ring.lean,Mathlib/Algebra/Order/Floor/Semiring.lean,Mathlib/Algebra/Order/Kleene.lean,Mathlib/Algebra/Order/Monoid/Unbundled/WithTop.lean,Mathlib/Algebra/Order/Round.lean,Mathlib/Algebra/Order/SuccPred/WithBot.lean,Mathlib/Algebra/Polynomial/Basic.lean,Mathlib/Algebra/Polynomial/Coeff.lean,Mathlib/Algebra/Polynomial/Degree/Definitions.lean,Mathlib/Algebra/Polynomial/Derivative.lean,Mathlib/Algebra/Polynomial/Eval/Defs.lean,Mathlib/Algebra/Quaternion.lean,Mathlib/Algebra/Ring/Center.lean,Mathlib/Algebra/Star/Basic.lean,Mathlib/Algebra/Star/SelfAdjoint.lean,Mathlib/AlgebraicTopology/FundamentalGroupoid/Basic.lean,Mathlib/Analysis/Complex/Basic.lean,Mathlib/Analysis/Normed/Group/Basic.lean,Mathlib/Analysis/RCLike/Basic.lean,Mathlib/Analysis/SpecialFunctions/Complex/Arg.lean,Mathlib/Analysis/SpecialFunctions/Complex/Log.lean,Mathlib/Analysis/SpecialFunctions/Gamma/Basic.lean,Mathlib/Analysis/SpecialFunctions/Pow/Complex.lean,Mathlib/Analysis/SpecialFunctions/Pow/NNReal.lean,Mathlib/Data/Complex/Basic.lean,Mathlib/Data/Complex/Norm.lean,Mathlib/Data/ENNReal/Basic.lean,Mathlib/Data/ENNReal/Real.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/Data/Int/Log.lean,Mathlib/Data/Matrix/ConjTranspose.lean,Mathlib/Data/Matrix/Diagonal.lean,Mathlib/Data/Matrix/Kronecker.lean,Mathlib/Data/Matrix/Mul.lean,Mathlib/Data/Matrix/Notation.lean,Mathlib/Data/NNRat/Defs.lean,Mathlib/Data/NNReal/Defs.lean,Mathlib/Data/Nat/Cast/Basic.lean,Mathlib/Data/Nat/Cast/Commute.lean,Mathlib/Data/Nat/Cast/Defs.lean,Mathlib/Data/Nat/Cast/Order/Basic.lean,Mathlib/Data/Nat/Cast/Order/Ring.lean,Mathlib/Data/Nat/Cast/Prod.lean,Mathlib/Data/Nat/Cast/Synonym.lean,Mathlib/Data/Nat/PartENat.lean,Mathlib/Data/Rat/Lemmas.lean,Mathlib/Data/Real/Hyperreal.lean,Mathlib/Data/Real/Irrational.lean,Mathlib/Data/ZMod/Basic.lean,Mathlib/Data/ZMod/IntUnitsPower.lean,Mathlib/Geometry/Manifold/IsManifold/Basic.lean,Mathlib/Geometry/Manifold/VectorField/Pullback.lean,Mathlib/LinearAlgebra/Dimension/Finrank.lean,Mathlib/LinearAlgebra/Matrix/PosDef.lean,Mathlib/MeasureTheory/Function/ConditionalExpectation/Basic.lean,Mathlib/NumberTheory/LucasLehmer.lean,Mathlib/NumberTheory/Padics/PadicNumbers.lean,Mathlib/NumberTheory/Zsqrtd/Basic.lean,Mathlib/Order/Filter/Germ/Basic.lean,Mathlib/RingTheory/Multiplicity.lean,Mathlib/SetTheory/Cardinal/Aleph.lean,Mathlib/SetTheory/Cardinal/Basic.lean,Mathlib/SetTheory/Cardinal/Continuum.lean,Mathlib/SetTheory/Cardinal/ENat.lean,Mathlib/SetTheory/Cardinal/Order.lean,Mathlib/SetTheory/Cardinal/ToNat.lean,Mathlib/SetTheory/Game/Birthday.lean,Mathlib/SetTheory/Game/Short.lean,Mathlib/SetTheory/Ordinal/Arithmetic.lean,Mathlib/SetTheory/Ordinal/Basic.lean,Mathlib/Tactic/ENatToNat.lean,Mathlib/Topology/Algebra/Module/LinearMap.lean,Mathlib/Topology/Algebra/SeparationQuotient/Basic.lean,Mathlib/Topology/ContinuousMap/Bounded/Normed.lean,Mathlib/Topology/Instances/ENNReal/Lemmas.lean 86 2 ['github-actions', 'leanprover-community-bot-assistant'] nobody
57-54259
1 month ago
57-54261
1 month ago
3-60152
3 days
23966 FR-vdash-bot
author:FR-vdash-bot
refactor: unbundle algebra from `{Seminormed, Normed}(Add)(Comm)Group` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) - [ ] depends on: #23621 - [ ] depends on: #23961 slow-typeclass-synthesis t-algebra t-analysis merge-conflict blocked-by-other-PR
label:t-algebra$
3233/2752 Archive/Imo/Imo1998Q2.lean,Counterexamples/LinearOrderWithPosMulPosEqZero.lean,Mathlib/Algebra/Module/ZLattice/Basic.lean,Mathlib/Algebra/Module/ZLattice/Covolume.lean,Mathlib/Algebra/Order/Field/Canonical.lean,Mathlib/Algebra/Order/Field/Rat.lean,Mathlib/Algebra/Order/Floor/Ring.lean,Mathlib/Algebra/Order/GroupWithZero/Canonical.lean,Mathlib/Algebra/Order/GroupWithZero/Finset.lean,Mathlib/Algebra/Order/Hom/Monoid.lean,Mathlib/Algebra/Order/Nonneg/Field.lean,Mathlib/Algebra/Order/Nonneg/Ring.lean,Mathlib/Algebra/Order/Ring/Nat.lean,Mathlib/Analysis/Analytic/Basic.lean,Mathlib/Analysis/Analytic/CPolynomial.lean,Mathlib/Analysis/Analytic/CPolynomialDef.lean,Mathlib/Analysis/Analytic/ChangeOrigin.lean,Mathlib/Analysis/Analytic/Composition.lean,Mathlib/Analysis/Analytic/Constructions.lean,Mathlib/Analysis/Analytic/Inverse.lean,Mathlib/Analysis/Analytic/IsolatedZeros.lean,Mathlib/Analysis/Analytic/IteratedFDeriv.lean,Mathlib/Analysis/Analytic/Linear.lean,Mathlib/Analysis/Analytic/Order.lean,Mathlib/Analysis/Analytic/Polynomial.lean,Mathlib/Analysis/Analytic/RadiusLiminf.lean,Mathlib/Analysis/Analytic/Uniqueness.lean,Mathlib/Analysis/Analytic/Within.lean,Mathlib/Analysis/Asymptotics/AsymptoticEquivalent.lean,Mathlib/Analysis/Asymptotics/Defs.lean,Mathlib/Analysis/Asymptotics/Lemmas.lean,Mathlib/Analysis/Asymptotics/SpecificAsymptotics.lean,Mathlib/Analysis/Asymptotics/TVS.lean,Mathlib/Analysis/Asymptotics/Theta.lean,Mathlib/Analysis/BoundedVariation.lean,Mathlib/Analysis/BoxIntegral/Basic.lean,Mathlib/Analysis/BoxIntegral/DivergenceTheorem.lean,Mathlib/Analysis/BoxIntegral/Integrability.lean,Mathlib/Analysis/BoxIntegral/Partition/Additive.lean,Mathlib/Analysis/BoxIntegral/Partition/Measure.lean,Mathlib/Analysis/CStarAlgebra/Basic.lean,Mathlib/Analysis/CStarAlgebra/CStarMatrix.lean,Mathlib/Analysis/CStarAlgebra/ContinuousLinearMap.lean,Mathlib/Analysis/CStarAlgebra/Matrix.lean,Mathlib/Analysis/CStarAlgebra/Module/Constructions.lean,Mathlib/Analysis/CStarAlgebra/Module/Defs.lean,Mathlib/Analysis/Calculus/AddTorsor/AffineMap.lean,Mathlib/Analysis/Calculus/AddTorsor/Coord.lean,Mathlib/Analysis/Calculus/BumpFunction/Basic.lean,Mathlib/Analysis/Calculus/BumpFunction/Convolution.lean,Mathlib/Analysis/Calculus/BumpFunction/FiniteDimension.lean,Mathlib/Analysis/Calculus/BumpFunction/InnerProduct.lean,Mathlib/Analysis/Calculus/BumpFunction/Normed.lean,Mathlib/Analysis/Calculus/Conformal/InnerProduct.lean,Mathlib/Analysis/Calculus/Conformal/NormedSpace.lean,Mathlib/Analysis/Calculus/ContDiff/Basic.lean,Mathlib/Analysis/Calculus/ContDiff/Bounds.lean,Mathlib/Analysis/Calculus/ContDiff/CPolynomial.lean,Mathlib/Analysis/Calculus/ContDiff/Defs.lean,Mathlib/Analysis/Calculus/ContDiff/FTaylorSeries.lean,Mathlib/Analysis/Calculus/ContDiff/FaaDiBruno.lean,Mathlib/Analysis/Calculus/ContDiff/FiniteDimension.lean,Mathlib/Analysis/Calculus/ContDiff/Operations.lean,Mathlib/Analysis/Calculus/ContDiff/RCLike.lean,Mathlib/Analysis/Calculus/ContDiff/WithLp.lean,Mathlib/Analysis/Calculus/DSlope.lean,Mathlib/Analysis/Calculus/Deriv/Abs.lean,Mathlib/Analysis/Calculus/Deriv/Add.lean,Mathlib/Analysis/Calculus/Deriv/AffineMap.lean,Mathlib/Analysis/Calculus/Deriv/Basic.lean,Mathlib/Analysis/Calculus/Deriv/Comp.lean,Mathlib/Analysis/Calculus/Deriv/Inv.lean,Mathlib/Analysis/Calculus/Deriv/Inverse.lean,Mathlib/Analysis/Calculus/Deriv/Linear.lean,Mathlib/Analysis/Calculus/Deriv/Mul.lean,Mathlib/Analysis/Calculus/Deriv/Prod.lean,Mathlib/Analysis/Calculus/Deriv/Shift.lean,Mathlib/Analysis/Calculus/Deriv/Slope.lean,Mathlib/Analysis/Calculus/Deriv/Star.lean,Mathlib/Analysis/Calculus/Deriv/Support.lean,Mathlib/Analysis/Calculus/Deriv/ZPow.lean,Mathlib/Analysis/Calculus/DiffContOnCl.lean,Mathlib/Analysis/Calculus/FDeriv/Add.lean,Mathlib/Analysis/Calculus/FDeriv/Analytic.lean,Mathlib/Analysis/Calculus/FDeriv/Basic.lean,Mathlib/Analysis/Calculus/FDeriv/Bilinear.lean,Mathlib/Analysis/Calculus/FDeriv/Comp.lean,Mathlib/Analysis/Calculus/FDeriv/Equiv.lean,Mathlib/Analysis/Calculus/FDeriv/Extend.lean,Mathlib/Analysis/Calculus/FDeriv/Linear.lean,Mathlib/Analysis/Calculus/FDeriv/Measurable.lean,Mathlib/Analysis/Calculus/FDeriv/Mul.lean,Mathlib/Analysis/Calculus/FDeriv/Norm.lean,Mathlib/Analysis/Calculus/FDeriv/Pi.lean,Mathlib/Analysis/Calculus/FDeriv/Prod.lean,Mathlib/Analysis/Calculus/FDeriv/RestrictScalars.lean,Mathlib/Analysis/Calculus/FDeriv/Star.lean,Mathlib/Analysis/Calculus/FDeriv/Symmetric.lean,Mathlib/Analysis/Calculus/FDeriv/WithLp.lean,Mathlib/Analysis/Calculus/FormalMultilinearSeries.lean 579 7 ['FR-vdash-bot', 'github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
56-17842
1 month ago
58-50701
1 month ago*
0-0
0 seconds*
24040 FR-vdash-bot
author:FR-vdash-bot
refactor: unbundle algebra from `(NonUnital){Seminormed, Normed}(Comm)Ring` --- - [ ] depends on: #23966 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) slow-typeclass-synthesis t-algebra t-analysis merge-conflict blocked-by-other-PR
label:t-algebra$
3775/3674 Archive/Imo/Imo1998Q2.lean,Counterexamples/LinearOrderWithPosMulPosEqZero.lean,Mathlib/Algebra/Algebra/RestrictScalars.lean,Mathlib/Algebra/Module/ZLattice/Basic.lean,Mathlib/Algebra/Module/ZLattice/Covolume.lean,Mathlib/Algebra/Order/Field/Canonical.lean,Mathlib/Algebra/Order/Field/Rat.lean,Mathlib/Algebra/Order/Floor/Ring.lean,Mathlib/Algebra/Order/GroupWithZero/Canonical.lean,Mathlib/Algebra/Order/GroupWithZero/Finset.lean,Mathlib/Algebra/Order/Hom/Monoid.lean,Mathlib/Algebra/Order/Nonneg/Field.lean,Mathlib/Algebra/Order/Nonneg/Ring.lean,Mathlib/Algebra/Order/Ring/Nat.lean,Mathlib/Analysis/Analytic/Basic.lean,Mathlib/Analysis/Analytic/CPolynomial.lean,Mathlib/Analysis/Analytic/CPolynomialDef.lean,Mathlib/Analysis/Analytic/ChangeOrigin.lean,Mathlib/Analysis/Analytic/Composition.lean,Mathlib/Analysis/Analytic/Constructions.lean,Mathlib/Analysis/Analytic/Inverse.lean,Mathlib/Analysis/Analytic/IsolatedZeros.lean,Mathlib/Analysis/Analytic/IteratedFDeriv.lean,Mathlib/Analysis/Analytic/Linear.lean,Mathlib/Analysis/Analytic/OfScalars.lean,Mathlib/Analysis/Analytic/Order.lean,Mathlib/Analysis/Analytic/Polynomial.lean,Mathlib/Analysis/Analytic/RadiusLiminf.lean,Mathlib/Analysis/Analytic/Uniqueness.lean,Mathlib/Analysis/Analytic/Within.lean,Mathlib/Analysis/Asymptotics/AsymptoticEquivalent.lean,Mathlib/Analysis/Asymptotics/Defs.lean,Mathlib/Analysis/Asymptotics/Lemmas.lean,Mathlib/Analysis/Asymptotics/SpecificAsymptotics.lean,Mathlib/Analysis/Asymptotics/TVS.lean,Mathlib/Analysis/Asymptotics/Theta.lean,Mathlib/Analysis/BoundedVariation.lean,Mathlib/Analysis/BoxIntegral/Basic.lean,Mathlib/Analysis/BoxIntegral/DivergenceTheorem.lean,Mathlib/Analysis/BoxIntegral/Integrability.lean,Mathlib/Analysis/BoxIntegral/Partition/Additive.lean,Mathlib/Analysis/BoxIntegral/Partition/Measure.lean,Mathlib/Analysis/CStarAlgebra/Basic.lean,Mathlib/Analysis/CStarAlgebra/CStarMatrix.lean,Mathlib/Analysis/CStarAlgebra/Classes.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Basic.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Instances.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Integral.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Isometric.lean,Mathlib/Analysis/CStarAlgebra/ContinuousLinearMap.lean,Mathlib/Analysis/CStarAlgebra/ContinuousMap.lean,Mathlib/Analysis/CStarAlgebra/Exponential.lean,Mathlib/Analysis/CStarAlgebra/GelfandDuality.lean,Mathlib/Analysis/CStarAlgebra/Matrix.lean,Mathlib/Analysis/CStarAlgebra/Module/Constructions.lean,Mathlib/Analysis/CStarAlgebra/Module/Defs.lean,Mathlib/Analysis/CStarAlgebra/Multiplier.lean,Mathlib/Analysis/CStarAlgebra/Spectrum.lean,Mathlib/Analysis/CStarAlgebra/Unitization.lean,Mathlib/Analysis/CStarAlgebra/lpSpace.lean,Mathlib/Analysis/Calculus/AddTorsor/AffineMap.lean,Mathlib/Analysis/Calculus/AddTorsor/Coord.lean,Mathlib/Analysis/Calculus/BumpFunction/Basic.lean,Mathlib/Analysis/Calculus/BumpFunction/Convolution.lean,Mathlib/Analysis/Calculus/BumpFunction/FiniteDimension.lean,Mathlib/Analysis/Calculus/BumpFunction/InnerProduct.lean,Mathlib/Analysis/Calculus/BumpFunction/Normed.lean,Mathlib/Analysis/Calculus/Conformal/InnerProduct.lean,Mathlib/Analysis/Calculus/Conformal/NormedSpace.lean,Mathlib/Analysis/Calculus/ContDiff/Basic.lean,Mathlib/Analysis/Calculus/ContDiff/Bounds.lean,Mathlib/Analysis/Calculus/ContDiff/CPolynomial.lean,Mathlib/Analysis/Calculus/ContDiff/Defs.lean,Mathlib/Analysis/Calculus/ContDiff/FTaylorSeries.lean,Mathlib/Analysis/Calculus/ContDiff/FaaDiBruno.lean,Mathlib/Analysis/Calculus/ContDiff/FiniteDimension.lean,Mathlib/Analysis/Calculus/ContDiff/Operations.lean,Mathlib/Analysis/Calculus/ContDiff/RCLike.lean,Mathlib/Analysis/Calculus/ContDiff/WithLp.lean,Mathlib/Analysis/Calculus/DSlope.lean,Mathlib/Analysis/Calculus/Deriv/Abs.lean,Mathlib/Analysis/Calculus/Deriv/Add.lean,Mathlib/Analysis/Calculus/Deriv/AffineMap.lean,Mathlib/Analysis/Calculus/Deriv/Basic.lean,Mathlib/Analysis/Calculus/Deriv/Comp.lean,Mathlib/Analysis/Calculus/Deriv/Inv.lean,Mathlib/Analysis/Calculus/Deriv/Inverse.lean,Mathlib/Analysis/Calculus/Deriv/Linear.lean,Mathlib/Analysis/Calculus/Deriv/Mul.lean,Mathlib/Analysis/Calculus/Deriv/Prod.lean,Mathlib/Analysis/Calculus/Deriv/Shift.lean,Mathlib/Analysis/Calculus/Deriv/Slope.lean,Mathlib/Analysis/Calculus/Deriv/Star.lean,Mathlib/Analysis/Calculus/Deriv/Support.lean,Mathlib/Analysis/Calculus/Deriv/ZPow.lean,Mathlib/Analysis/Calculus/DiffContOnCl.lean,Mathlib/Analysis/Calculus/FDeriv/Add.lean,Mathlib/Analysis/Calculus/FDeriv/Analytic.lean,Mathlib/Analysis/Calculus/FDeriv/Basic.lean,Mathlib/Analysis/Calculus/FDeriv/Bilinear.lean 630 n/a ['FR-vdash-bot', 'github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
56-17720
1 month ago
unknown
unknown
16314 FR-vdash-bot
author:FR-vdash-bot
chore(Data/Quot): deprecate `ind*'` APIs --- - [x] depends on: #16264 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data merge-conflict 247/287 Counterexamples/CliffordAlgebraNotInjective.lean,Mathlib/Algebra/Colimit/Module.lean,Mathlib/Algebra/Lie/Quotient.lean,Mathlib/Algebra/Module/Torsion.lean,Mathlib/Algebra/RingQuot.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Angle.lean,Mathlib/CategoryTheory/ConnectedComponents.lean,Mathlib/CategoryTheory/Subobject/Basic.lean,Mathlib/CategoryTheory/Subobject/FactorThru.lean,Mathlib/CategoryTheory/Subobject/Lattice.lean,Mathlib/Computability/Reduce.lean,Mathlib/Computability/Tape.lean,Mathlib/Data/List/Cycle.lean,Mathlib/Data/Multiset/MapFold.lean,Mathlib/Data/Multiset/ZeroCons.lean,Mathlib/Data/Quot.lean,Mathlib/Data/Setoid/Basic.lean,Mathlib/Data/Setoid/Partition.lean,Mathlib/FieldTheory/Fixed.lean,Mathlib/GroupTheory/Complement.lean,Mathlib/GroupTheory/Congruence/Basic.lean,Mathlib/GroupTheory/Congruence/Defs.lean,Mathlib/GroupTheory/Congruence/Hom.lean,Mathlib/GroupTheory/Coset/Basic.lean,Mathlib/GroupTheory/Coset/Defs.lean,Mathlib/GroupTheory/FreeAbelianGroup.lean,Mathlib/GroupTheory/GroupAction/Basic.lean,Mathlib/GroupTheory/GroupAction/Defs.lean,Mathlib/GroupTheory/GroupAction/Quotient.lean,Mathlib/GroupTheory/Index.lean,Mathlib/GroupTheory/MonoidLocalization/Basic.lean,Mathlib/GroupTheory/PGroup.lean,Mathlib/GroupTheory/Perm/Cycle/Concrete.lean,Mathlib/GroupTheory/PresentedGroup.lean,Mathlib/GroupTheory/QuotientGroup/Basic.lean,Mathlib/GroupTheory/QuotientGroup/Defs.lean,Mathlib/GroupTheory/SchurZassenhaus.lean,Mathlib/GroupTheory/Sylow.lean,Mathlib/LinearAlgebra/Alternating/DomCoprod.lean,Mathlib/LinearAlgebra/Projectivization/Basic.lean,Mathlib/LinearAlgebra/Quotient/Basic.lean,Mathlib/LinearAlgebra/Quotient/Defs.lean,Mathlib/MeasureTheory/Function/AEEqFun.lean,Mathlib/NumberTheory/Padics/PadicNumbers.lean,Mathlib/NumberTheory/RamificationInertia/Basic.lean,Mathlib/Order/Antisymmetrization.lean,Mathlib/Order/Category/PartOrd.lean,Mathlib/Order/Filter/Germ/Basic.lean,Mathlib/RepresentationTheory/GroupCohomology/Hilbert90.lean,Mathlib/RingTheory/AdicCompletion/Algebra.lean,Mathlib/RingTheory/AdicCompletion/Basic.lean,Mathlib/RingTheory/AdicCompletion/Functoriality.lean,Mathlib/RingTheory/AdjoinRoot.lean,Mathlib/RingTheory/Congruence/Basic.lean,Mathlib/RingTheory/Flat/FaithfullyFlat/Basic.lean,Mathlib/RingTheory/GradedAlgebra/HomogeneousLocalization.lean,Mathlib/RingTheory/Ideal/Cotangent.lean,Mathlib/RingTheory/Ideal/Norm/AbsNorm.lean,Mathlib/RingTheory/Ideal/Quotient/Basic.lean,Mathlib/RingTheory/Ideal/Quotient/Defs.lean,Mathlib/RingTheory/Ideal/Quotient/Operations.lean,Mathlib/RingTheory/Valuation/Quotient.lean,Mathlib/Topology/Algebra/Group/TopologicalAbelianization.lean,Mathlib/Topology/Algebra/InfiniteSum/Module.lean,Mathlib/Topology/Separation/Basic.lean 65 4 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
55-49253
1 month ago
55-49255
1 month ago
55-52030
55 days
23211 Parcly-Taxel
author:Parcly-Taxel
chore: automatically deprime common `induction'` uses Replace `induction'` with `induction` for the following targets: ```python rep_dict = {("Nat", "~", 2): [("zero", 0), ("succ", 2)], ("Nat", "strong_induction_on", 1): [("h", 2)], ("Nat", "case_strong_induction_on", 2): [("hz", 0), ("hi", 2)], ("Nat", "le_induction", 2): [("base", 0), ("succ", 3)], ("List", "~", 2): [("nil", 0), ("cons", 3)], ("List", "reverseRecOn", 2): [("nil", 0), ("append_singleton", 3)], ("Multiset", "induction_on", 2): [("empty", 0), ("cons", 3)], ("Finset", "induction", 2): [("empty", 0), ("@insert", 4)], ("Finset", "induction_on", 2): [("empty", 0), ("@insert", 4)], ("MvPolynomial", "induction_on'", 2): [("monomial", 2), ("add", 4)], ("MvPolynomial", "induction_on", 3): [("C", 1), ("add", 4), ("mul_X", 3)]} ``` The script and the data file used can be found [here](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/The.20plan.20to.20remove.20induction'/near/508218834). tech debt merge-conflict 2189/1565 Archive/Imo/Imo1977Q6.lean,Archive/Imo/Imo2006Q5.lean,Archive/Imo/Imo2013Q1.lean,Archive/Imo/Imo2013Q5.lean,Archive/Imo/Imo2019Q4.lean,Archive/Imo/Imo2024Q1.lean,Archive/MiuLanguage/DecisionSuf.lean,Archive/Sensitivity.lean,Archive/Wiedijk100Theorems/FriendshipGraphs.lean,Archive/Wiedijk100Theorems/Partition.lean,Mathlib/Algebra/Algebra/Subalgebra/Lattice.lean,Mathlib/Algebra/BigOperators/Group/List/Lemmas.lean,Mathlib/Algebra/Group/Conj.lean,Mathlib/Algebra/Group/ForwardDiff.lean,Mathlib/Algebra/Group/Pointwise/Finset/Basic.lean,Mathlib/Algebra/Group/Pointwise/Set/BigOperators.lean,Mathlib/Algebra/Group/Pointwise/Set/Finite.lean,Mathlib/Algebra/Group/Pointwise/Set/ListOfFn.lean,Mathlib/Algebra/Lie/Solvable.lean,Mathlib/Algebra/Module/PID.lean,Mathlib/Algebra/Order/BigOperators/Group/List.lean,Mathlib/Algebra/Order/CauSeq/BigOperators.lean,Mathlib/Algebra/Order/Group/Multiset.lean,Mathlib/Algebra/Polynomial/BigOperators.lean,Mathlib/Algebra/Polynomial/Degree/Lemmas.lean,Mathlib/Algebra/Polynomial/Derivative.lean,Mathlib/Algebra/Polynomial/EraseLead.lean,Mathlib/Algebra/Polynomial/Eval/Defs.lean,Mathlib/Algebra/Polynomial/HasseDeriv.lean,Mathlib/Algebra/Ring/Subring/Basic.lean,Mathlib/Algebra/Tropical/BigOperators.lean,Mathlib/AlgebraicTopology/DoldKan/Decomposition.lean,Mathlib/AlgebraicTopology/DoldKan/Degeneracies.lean,Mathlib/AlgebraicTopology/DoldKan/Projections.lean,Mathlib/Analysis/Analytic/Composition.lean,Mathlib/Analysis/Analytic/Constructions.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/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/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/Log/Base.lean,Mathlib/Analysis/SpecialFunctions/Pow/Deriv.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/EulerSineProd.lean,Mathlib/CategoryTheory/ComposableArrows.lean,Mathlib/CategoryTheory/Extensive.lean,Mathlib/CategoryTheory/Filtered/Basic.lean,Mathlib/CategoryTheory/Limits/VanKampen.lean,Mathlib/CategoryTheory/Triangulated/TStructure/Basic.lean,Mathlib/Computability/Ackermann.lean,Mathlib/Computability/DFA.lean,Mathlib/Computability/EpsilonNFA.lean,Mathlib/Computability/Language.lean,Mathlib/Computability/NFA.lean,Mathlib/Computability/Partrec.lean,Mathlib/Computability/PartrecCode.lean,Mathlib/Computability/PostTuringMachine.lean,Mathlib/Computability/Primrec.lean,Mathlib/Computability/RegularExpressions.lean,Mathlib/Computability/TMConfig.lean,Mathlib/Computability/TMToPartrec.lean,Mathlib/Computability/Tape.lean,Mathlib/Control/LawfulFix.lean,Mathlib/Data/Complex/Exponential.lean,Mathlib/Data/Countable/Basic.lean,Mathlib/Data/DFinsupp/Defs.lean,Mathlib/Data/DFinsupp/WellFounded.lean,Mathlib/Data/Fin/Tuple/Basic.lean,Mathlib/Data/Fin/Tuple/NatAntidiagonal.lean,Mathlib/Data/Finmap.lean,Mathlib/Data/Finset/Fold.lean,Mathlib/Data/Finset/Image.lean,Mathlib/Data/Finset/Lattice/Fold.lean,Mathlib/Data/Finset/Lattice/Lemmas.lean,Mathlib/Data/Finset/Lattice/Pi.lean,Mathlib/Data/Finset/Max.lean,Mathlib/Data/Finset/NAry.lean,Mathlib/Data/Finset/NoncommProd.lean,Mathlib/Data/Finset/Sym.lean,Mathlib/Data/Finsupp/BigOperators.lean,Mathlib/Data/Fintype/Basic.lean,Mathlib/Data/Fintype/Card.lean,Mathlib/Data/Fintype/EquivFin.lean,Mathlib/Data/Fintype/Fin.lean 283 2 ['github-actions', 'leanprover-community-bot-assistant'] nobody
55-47427
1 month ago
55-47429
1 month ago
10-65025
10 days
13795 FR-vdash-bot
author:FR-vdash-bot
perf(Algebra/{Group, GroupWithZero, Ring}/InjSurj): reduce everything --- - [ ] depends on: #15192 - [ ] depends on: #15476 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict
label:t-algebra$
340/194 Mathlib/Algebra/Equiv/TransferInstance.lean,Mathlib/Algebra/Group/InjSurj.lean,Mathlib/Algebra/GroupWithZero/Action/Defs.lean,Mathlib/Algebra/GroupWithZero/Action/End.lean,Mathlib/Algebra/GroupWithZero/InjSurj.lean,Mathlib/Algebra/Module/Defs.lean,Mathlib/Algebra/Module/RingHom.lean,Mathlib/Algebra/Ring/InjSurj.lean,scripts/noshake.json 9 35 ['FR-vdash-bot', 'MichaelStollBayreuth', 'eric-wieser', 'github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mattrobball'] nobody
55-41568
1 month ago
55-41570
1 month ago
52-31623
52 days
23509 eric-wieser
author:eric-wieser
refactor: Make ENNReal an abbrev The `Coe` instance becomes `CoeTC` to match what we do for `WithTop` (such that the priority kicks in) Probably we could have both copies and things would be ok. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) This includes part of #23750 t-data merge-conflict 22/66 Mathlib/Data/ENNReal/Basic.lean,Mathlib/Data/ENNReal/BigOperators.lean,Mathlib/Data/ENNReal/Operations.lean,Mathlib/MeasureTheory/Integral/SetToL1.lean,Mathlib/MeasureTheory/Measure/Sub.lean,Mathlib/MeasureTheory/Measure/TightNormed.lean,Mathlib/Topology/MetricSpace/PartitionOfUnity.lean 7 22 ['eric-wieser', 'github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'leanprover-community-mathlib4-bot', 'mattrobball', 'urkud'] nobody
55-32906
1 month ago
55-32908
1 month ago
14-12910
14 days
24060 eric-wieser
author:eric-wieser
chore(MeasureTheory): use `0` instead of `const _ 0` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-measure-probability merge-conflict 30/20 Mathlib/MeasureTheory/Function/SimpleFunc.lean,Mathlib/MeasureTheory/Function/SimpleFuncDense.lean,Mathlib/MeasureTheory/Function/SimpleFuncDenseLp.lean,Mathlib/MeasureTheory/Integral/Bochner/VitaliCaratheodory.lean,Mathlib/MeasureTheory/Integral/Lebesgue/Countable.lean,Mathlib/MeasureTheory/Integral/SetToL1.lean,Mathlib/Probability/StrongLaw.lean 7 2 ['github-actions', 'leanprover-community-bot-assistant'] nobody
55-22601
1 month ago
55-22603
1 month ago
0-0
0 seconds
24058 FR-vdash-bot
author:FR-vdash-bot
refactor: unbundle algebra from `*NormedField` --- - [ ] depends on: #24040 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) slow-typeclass-synthesis t-algebra t-analysis merge-conflict blocked-by-other-PR
label:t-algebra$
4602/4346 Archive/Hairer.lean,Archive/Imo/Imo1998Q2.lean,Counterexamples/LinearOrderWithPosMulPosEqZero.lean,Mathlib/Algebra/Algebra/RestrictScalars.lean,Mathlib/Algebra/Module/ZLattice/Basic.lean,Mathlib/Algebra/Module/ZLattice/Covolume.lean,Mathlib/Algebra/Order/Field/Canonical.lean,Mathlib/Algebra/Order/Field/Rat.lean,Mathlib/Algebra/Order/Floor/Ring.lean,Mathlib/Algebra/Order/GroupWithZero/Canonical.lean,Mathlib/Algebra/Order/GroupWithZero/Finset.lean,Mathlib/Algebra/Order/Hom/Monoid.lean,Mathlib/Algebra/Order/Nonneg/Field.lean,Mathlib/Algebra/Order/Nonneg/Ring.lean,Mathlib/Algebra/Order/Ring/Nat.lean,Mathlib/Analysis/Analytic/Basic.lean,Mathlib/Analysis/Analytic/CPolynomial.lean,Mathlib/Analysis/Analytic/CPolynomialDef.lean,Mathlib/Analysis/Analytic/ChangeOrigin.lean,Mathlib/Analysis/Analytic/Composition.lean,Mathlib/Analysis/Analytic/Constructions.lean,Mathlib/Analysis/Analytic/Inverse.lean,Mathlib/Analysis/Analytic/IsolatedZeros.lean,Mathlib/Analysis/Analytic/IteratedFDeriv.lean,Mathlib/Analysis/Analytic/Linear.lean,Mathlib/Analysis/Analytic/OfScalars.lean,Mathlib/Analysis/Analytic/Order.lean,Mathlib/Analysis/Analytic/Polynomial.lean,Mathlib/Analysis/Analytic/RadiusLiminf.lean,Mathlib/Analysis/Analytic/Uniqueness.lean,Mathlib/Analysis/Analytic/Within.lean,Mathlib/Analysis/Asymptotics/AsymptoticEquivalent.lean,Mathlib/Analysis/Asymptotics/Defs.lean,Mathlib/Analysis/Asymptotics/Lemmas.lean,Mathlib/Analysis/Asymptotics/SpecificAsymptotics.lean,Mathlib/Analysis/Asymptotics/SuperpolynomialDecay.lean,Mathlib/Analysis/Asymptotics/TVS.lean,Mathlib/Analysis/Asymptotics/Theta.lean,Mathlib/Analysis/BoundedVariation.lean,Mathlib/Analysis/BoxIntegral/Basic.lean,Mathlib/Analysis/BoxIntegral/DivergenceTheorem.lean,Mathlib/Analysis/BoxIntegral/Integrability.lean,Mathlib/Analysis/BoxIntegral/Partition/Additive.lean,Mathlib/Analysis/BoxIntegral/Partition/Measure.lean,Mathlib/Analysis/CStarAlgebra/Basic.lean,Mathlib/Analysis/CStarAlgebra/CStarMatrix.lean,Mathlib/Analysis/CStarAlgebra/Classes.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Basic.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Instances.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Integral.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Isometric.lean,Mathlib/Analysis/CStarAlgebra/ContinuousLinearMap.lean,Mathlib/Analysis/CStarAlgebra/ContinuousMap.lean,Mathlib/Analysis/CStarAlgebra/Exponential.lean,Mathlib/Analysis/CStarAlgebra/GelfandDuality.lean,Mathlib/Analysis/CStarAlgebra/Matrix.lean,Mathlib/Analysis/CStarAlgebra/Module/Constructions.lean,Mathlib/Analysis/CStarAlgebra/Module/Defs.lean,Mathlib/Analysis/CStarAlgebra/Multiplier.lean,Mathlib/Analysis/CStarAlgebra/Spectrum.lean,Mathlib/Analysis/CStarAlgebra/Unitization.lean,Mathlib/Analysis/CStarAlgebra/lpSpace.lean,Mathlib/Analysis/Calculus/AddTorsor/AffineMap.lean,Mathlib/Analysis/Calculus/AddTorsor/Coord.lean,Mathlib/Analysis/Calculus/BumpFunction/Basic.lean,Mathlib/Analysis/Calculus/BumpFunction/Convolution.lean,Mathlib/Analysis/Calculus/BumpFunction/FiniteDimension.lean,Mathlib/Analysis/Calculus/BumpFunction/InnerProduct.lean,Mathlib/Analysis/Calculus/BumpFunction/Normed.lean,Mathlib/Analysis/Calculus/Conformal/InnerProduct.lean,Mathlib/Analysis/Calculus/Conformal/NormedSpace.lean,Mathlib/Analysis/Calculus/ContDiff/Basic.lean,Mathlib/Analysis/Calculus/ContDiff/Bounds.lean,Mathlib/Analysis/Calculus/ContDiff/CPolynomial.lean,Mathlib/Analysis/Calculus/ContDiff/Defs.lean,Mathlib/Analysis/Calculus/ContDiff/FTaylorSeries.lean,Mathlib/Analysis/Calculus/ContDiff/FaaDiBruno.lean,Mathlib/Analysis/Calculus/ContDiff/FiniteDimension.lean,Mathlib/Analysis/Calculus/ContDiff/Operations.lean,Mathlib/Analysis/Calculus/ContDiff/RCLike.lean,Mathlib/Analysis/Calculus/ContDiff/WithLp.lean,Mathlib/Analysis/Calculus/DSlope.lean,Mathlib/Analysis/Calculus/Deriv/Abs.lean,Mathlib/Analysis/Calculus/Deriv/Add.lean,Mathlib/Analysis/Calculus/Deriv/AffineMap.lean,Mathlib/Analysis/Calculus/Deriv/Basic.lean,Mathlib/Analysis/Calculus/Deriv/Comp.lean,Mathlib/Analysis/Calculus/Deriv/Inv.lean,Mathlib/Analysis/Calculus/Deriv/Inverse.lean,Mathlib/Analysis/Calculus/Deriv/Linear.lean,Mathlib/Analysis/Calculus/Deriv/Mul.lean,Mathlib/Analysis/Calculus/Deriv/Pi.lean,Mathlib/Analysis/Calculus/Deriv/Polynomial.lean,Mathlib/Analysis/Calculus/Deriv/Pow.lean,Mathlib/Analysis/Calculus/Deriv/Prod.lean,Mathlib/Analysis/Calculus/Deriv/Shift.lean,Mathlib/Analysis/Calculus/Deriv/Slope.lean,Mathlib/Analysis/Calculus/Deriv/Star.lean,Mathlib/Analysis/Calculus/Deriv/Support.lean,Mathlib/Analysis/Calculus/Deriv/ZPow.lean 665 7 ['FR-vdash-bot', 'github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
55-12511
1 month ago
55-74730
1 month ago*
0-0
0 seconds*
11455 adomani
author:adomani
fix: unsqueeze simp, re Yaël's comments on #11259 This PR reverts/simplifies some of the "squeeze `simp`" changes in #11259. See #11259 for context. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author 3/6 Mathlib/Algebra/Group/Conj.lean,Mathlib/Data/Seq/WSeq.lean 2 8 ['Ruben-VandeVelde', 'YaelDillies', 'grunweg', 'loefflerd', 'robertylewis', 'urkud'] nobody
54-80906
1 month ago
325-21096
10 months ago
91-14162
91 days
8453 FR-vdash-bot
author:FR-vdash-bot
chore(MeasureTheory): Golf, speed up --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-measure-probability merge-conflict 29/42 Mathlib/MeasureTheory/Integral/DivergenceTheorem.lean,Mathlib/MeasureTheory/Measure/FiniteMeasure.lean,Mathlib/MeasureTheory/Measure/Haar/Unique.lean,Mathlib/MeasureTheory/Measure/MeasureSpace.lean,Mathlib/MeasureTheory/Measure/Portmanteau.lean,Mathlib/MeasureTheory/Measure/ProbabilityMeasure.lean,Mathlib/MeasureTheory/Measure/Regular.lean,Mathlib/Probability/ConditionalProbability.lean,Mathlib/Probability/Kernel/Condexp.lean 9 14 ['FR-vdash-bot', 'YaelDillies', 'eric-wieser', 'github-actions', 'grunweg', 'leanprover-bot'] nobody
54-80825
1 month ago
335-23470
11 months ago
16-40723
16 days
7325 eric-wieser
author:eric-wieser
chore: use preimageIso instead of defeq abuse for InducedCategory This makes a few things slightly more verbose, but the type casts are now explicit in those places. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory awaiting-CI merge-conflict 22/21 Mathlib/CategoryTheory/EssentialImage.lean,Mathlib/CategoryTheory/Monoidal/Braided.lean,Mathlib/CategoryTheory/Monoidal/Subcategory.lean 3 1 ['grunweg'] nobody
54-80785
1 month ago
335-23470
11 months ago
0-0
0 seconds
7874 FR-vdash-bot
author:FR-vdash-bot
chore: make `IsScalarTower A A B` and `IsScalarTower A B B` higher priority --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) slow-typeclass-synthesis t-algebra awaiting-CI merge-conflict
label:t-algebra$
10/9 Mathlib/Algebra/Algebra/Defs.lean,Mathlib/Algebra/Group/Action/Defs.lean,Mathlib/Data/Rat/Cast/Defs.lean,Mathlib/GroupTheory/GroupAction/Ring.lean 4 3 ['FR-vdash-bot', 'grunweg', 'leanprover-bot'] nobody
54-80760
1 month ago
325-21355
10 months ago
0-0
0 seconds
5952 eric-wieser
author:eric-wieser
feat: add Qq wrappers for ToExpr --- - [ ] depends on: #6699 (to appease the linter) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-CI t-meta merge-conflict 247/150 Mathlib/Data/Fin/Basic.lean,Mathlib/Data/Fin/VecNotation.lean,Mathlib/Data/Matrix/Notation.lean,Mathlib/Tactic/DeriveToExpr.lean,Mathlib/Tactic/FBinop.lean,Mathlib/Tactic/ToExpr.lean,Mathlib/Util/Qq.lean,test/DeriveToExpr.lean,test/vec_notation.lean 9 7 ['eric-wieser', 'gebner', 'grunweg', 'leanprover-community-mathlib4-bot'] nobody
54-80586
1 month ago
335-23470
11 months ago
29-67421
29 days
15483 FR-vdash-bot
author:FR-vdash-bot
chore(GroupTheory/Coset): reduce defeq abuse --- - [x] depends on: #15482 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict
label:t-algebra$
114/60 Mathlib/GroupTheory/Commensurable.lean,Mathlib/GroupTheory/Coset.lean,Mathlib/GroupTheory/QuotientGroup.lean,Mathlib/LinearAlgebra/Alternating/DomCoprod.lean,Mathlib/MeasureTheory/Measure/Haar/Quotient.lean,Mathlib/Topology/Algebra/Group/Compact.lean 6 14 ['FR-vdash-bot', 'eric-wieser', 'github-actions', 'grunweg', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'mattrobball', 'mergify', 'urkud'] nobody
54-80546
1 month ago
303-32476
9 months ago
4-79214
4 days
16594 FR-vdash-bot
author:FR-vdash-bot
perf: reorder `extends` and remove some instances in algebra hierarchy --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) slow-typeclass-synthesis t-algebra merge-conflict
label:t-algebra$
240/92 Mathlib.lean,Mathlib/Algebra/Algebra/Hom.lean,Mathlib/Algebra/Associated/Basic.lean,Mathlib/Algebra/BigOperators/Ring/List.lean,Mathlib/Algebra/Field/Defs.lean,Mathlib/Algebra/GCDMonoid/Basic.lean,Mathlib/Algebra/Group/Defs.lean,Mathlib/Algebra/Group/Ext.lean,Mathlib/Algebra/Group/Opposite.lean,Mathlib/Algebra/Group/Prod.lean,Mathlib/Algebra/GroupWithZero/Defs.lean,Mathlib/Algebra/GroupWithZero/Prod.lean,Mathlib/Algebra/Homology/Embedding/Basic.lean,Mathlib/Algebra/Order/AddGroupWithTop.lean,Mathlib/Algebra/Order/Field/Canonical/Defs.lean,Mathlib/Algebra/Order/Field/Defs.lean,Mathlib/Algebra/Order/Group/Unbundled/Abs.lean,Mathlib/Algebra/Order/GroupWithZero/Canonical.lean,Mathlib/Algebra/Order/Ring/Canonical.lean,Mathlib/Algebra/Order/Ring/Defs.lean,Mathlib/Algebra/Polynomial/Roots.lean,Mathlib/Algebra/Quaternion.lean,Mathlib/Algebra/Ring/Defs.lean,Mathlib/Algebra/Ring/Ext.lean,Mathlib/Algebra/Ring/InjSurj.lean,Mathlib/Algebra/Ring/Rat.lean,Mathlib/Algebra/Ring/SumsOfSquares.lean,Mathlib/Algebra/Tropical/Basic.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Order.lean,Mathlib/Analysis/InnerProductSpace/Symmetric.lean,Mathlib/CategoryTheory/Preadditive/FunctorCategory.lean,Mathlib/Data/Finset/NoncommProd.lean,Mathlib/Data/Int/Cast/Defs.lean,Mathlib/FieldTheory/IsAlgClosed/AlgebraicClosure.lean,Mathlib/FieldTheory/SplittingField/Construction.lean,Mathlib/GroupTheory/Congruence/Basic.lean,Mathlib/GroupTheory/MonoidLocalization/MonoidWithZero.lean,Mathlib/GroupTheory/Torsion.lean,Mathlib/LinearAlgebra/LinearPMap.lean,Mathlib/LinearAlgebra/TensorProduct/Basic.lean,Mathlib/Order/Filter/Germ/Basic.lean,Mathlib/Order/Interval/Finset/Box.lean,Mathlib/RingTheory/Bialgebra/Hom.lean,Mathlib/RingTheory/Coalgebra/Hom.lean,Mathlib/RingTheory/Ideal/Quotient.lean,Mathlib/RingTheory/Perfection.lean,Mathlib/RingTheory/TensorProduct/Basic.lean,Mathlib/RingTheory/TensorProduct/MvPolynomial.lean,Mathlib/Util/NoInstances.lean,scripts/noshake.json 50 8 ['FR-vdash-bot', 'github-actions', 'grunweg', 'leanprover-bot'] nobody
54-80322
1 month ago
259-33469
8 months ago
14-58900
14 days
24106 FR-vdash-bot
author:FR-vdash-bot
refactor: unbundle algebra from `*CStarAlgebra` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) - [ ] depends on: #24058 slow-typeclass-synthesis t-algebra t-analysis merge-conflict blocked-by-other-PR
label:t-algebra$
4702/4459 Archive/Hairer.lean,Archive/Imo/Imo1998Q2.lean,Counterexamples/LinearOrderWithPosMulPosEqZero.lean,Mathlib/Algebra/Algebra/RestrictScalars.lean,Mathlib/Algebra/Module/ZLattice/Basic.lean,Mathlib/Algebra/Module/ZLattice/Covolume.lean,Mathlib/Algebra/Order/Field/Canonical.lean,Mathlib/Algebra/Order/Field/Rat.lean,Mathlib/Algebra/Order/Floor/Ring.lean,Mathlib/Algebra/Order/GroupWithZero/Canonical.lean,Mathlib/Algebra/Order/GroupWithZero/Finset.lean,Mathlib/Algebra/Order/Hom/Monoid.lean,Mathlib/Algebra/Order/Nonneg/Field.lean,Mathlib/Algebra/Order/Nonneg/Ring.lean,Mathlib/Algebra/Order/Ring/Nat.lean,Mathlib/Analysis/Analytic/Basic.lean,Mathlib/Analysis/Analytic/CPolynomial.lean,Mathlib/Analysis/Analytic/CPolynomialDef.lean,Mathlib/Analysis/Analytic/ChangeOrigin.lean,Mathlib/Analysis/Analytic/Composition.lean,Mathlib/Analysis/Analytic/Constructions.lean,Mathlib/Analysis/Analytic/Inverse.lean,Mathlib/Analysis/Analytic/IsolatedZeros.lean,Mathlib/Analysis/Analytic/IteratedFDeriv.lean,Mathlib/Analysis/Analytic/Linear.lean,Mathlib/Analysis/Analytic/OfScalars.lean,Mathlib/Analysis/Analytic/Order.lean,Mathlib/Analysis/Analytic/Polynomial.lean,Mathlib/Analysis/Analytic/RadiusLiminf.lean,Mathlib/Analysis/Analytic/Uniqueness.lean,Mathlib/Analysis/Analytic/Within.lean,Mathlib/Analysis/Asymptotics/AsymptoticEquivalent.lean,Mathlib/Analysis/Asymptotics/Defs.lean,Mathlib/Analysis/Asymptotics/Lemmas.lean,Mathlib/Analysis/Asymptotics/SpecificAsymptotics.lean,Mathlib/Analysis/Asymptotics/SuperpolynomialDecay.lean,Mathlib/Analysis/Asymptotics/TVS.lean,Mathlib/Analysis/Asymptotics/Theta.lean,Mathlib/Analysis/BoundedVariation.lean,Mathlib/Analysis/BoxIntegral/Basic.lean,Mathlib/Analysis/BoxIntegral/DivergenceTheorem.lean,Mathlib/Analysis/BoxIntegral/Integrability.lean,Mathlib/Analysis/BoxIntegral/Partition/Additive.lean,Mathlib/Analysis/BoxIntegral/Partition/Measure.lean,Mathlib/Analysis/CStarAlgebra/ApproximateUnit.lean,Mathlib/Analysis/CStarAlgebra/Basic.lean,Mathlib/Analysis/CStarAlgebra/CStarMatrix.lean,Mathlib/Analysis/CStarAlgebra/Classes.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Basic.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Instances.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Integral.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Isometric.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Order.lean,Mathlib/Analysis/CStarAlgebra/ContinuousLinearMap.lean,Mathlib/Analysis/CStarAlgebra/ContinuousMap.lean,Mathlib/Analysis/CStarAlgebra/Exponential.lean,Mathlib/Analysis/CStarAlgebra/GelfandDuality.lean,Mathlib/Analysis/CStarAlgebra/Hom.lean,Mathlib/Analysis/CStarAlgebra/Matrix.lean,Mathlib/Analysis/CStarAlgebra/Module/Constructions.lean,Mathlib/Analysis/CStarAlgebra/Module/Defs.lean,Mathlib/Analysis/CStarAlgebra/Multiplier.lean,Mathlib/Analysis/CStarAlgebra/PositiveLinearMap.lean,Mathlib/Analysis/CStarAlgebra/SpecialFunctions/PosPart.lean,Mathlib/Analysis/CStarAlgebra/Spectrum.lean,Mathlib/Analysis/CStarAlgebra/Unitization.lean,Mathlib/Analysis/CStarAlgebra/lpSpace.lean,Mathlib/Analysis/Calculus/AddTorsor/AffineMap.lean,Mathlib/Analysis/Calculus/AddTorsor/Coord.lean,Mathlib/Analysis/Calculus/BumpFunction/Basic.lean,Mathlib/Analysis/Calculus/BumpFunction/Convolution.lean,Mathlib/Analysis/Calculus/BumpFunction/FiniteDimension.lean,Mathlib/Analysis/Calculus/BumpFunction/InnerProduct.lean,Mathlib/Analysis/Calculus/BumpFunction/Normed.lean,Mathlib/Analysis/Calculus/Conformal/InnerProduct.lean,Mathlib/Analysis/Calculus/Conformal/NormedSpace.lean,Mathlib/Analysis/Calculus/ContDiff/Basic.lean,Mathlib/Analysis/Calculus/ContDiff/Bounds.lean,Mathlib/Analysis/Calculus/ContDiff/CPolynomial.lean,Mathlib/Analysis/Calculus/ContDiff/Defs.lean,Mathlib/Analysis/Calculus/ContDiff/FTaylorSeries.lean,Mathlib/Analysis/Calculus/ContDiff/FaaDiBruno.lean,Mathlib/Analysis/Calculus/ContDiff/FiniteDimension.lean,Mathlib/Analysis/Calculus/ContDiff/Operations.lean,Mathlib/Analysis/Calculus/ContDiff/RCLike.lean,Mathlib/Analysis/Calculus/ContDiff/WithLp.lean,Mathlib/Analysis/Calculus/DSlope.lean,Mathlib/Analysis/Calculus/Deriv/Abs.lean,Mathlib/Analysis/Calculus/Deriv/Add.lean,Mathlib/Analysis/Calculus/Deriv/AffineMap.lean,Mathlib/Analysis/Calculus/Deriv/Basic.lean,Mathlib/Analysis/Calculus/Deriv/Comp.lean,Mathlib/Analysis/Calculus/Deriv/Inv.lean,Mathlib/Analysis/Calculus/Deriv/Inverse.lean,Mathlib/Analysis/Calculus/Deriv/Linear.lean,Mathlib/Analysis/Calculus/Deriv/Mul.lean,Mathlib/Analysis/Calculus/Deriv/Pi.lean,Mathlib/Analysis/Calculus/Deriv/Polynomial.lean,Mathlib/Analysis/Calculus/Deriv/Pow.lean,Mathlib/Analysis/Calculus/Deriv/Prod.lean 670 5 ['FR-vdash-bot', 'github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
54-52052
1 month ago
54-54359
1 month ago*
0-0
0 seconds*
13780 adomani
author:adomani
deprecate injective --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict 31/9 .github/workflows/bors.yml,.github/workflows/build.yml,.github/workflows/build.yml.in,.github/workflows/build_fork.yml,Mathlib/Init/Function.lean,lake-manifest.json,lakefile.lean 7 2 ['github-actions', 'grunweg'] nobody
54-47836
1 month ago
350-31180
11 months ago
0-0
0 seconds
11297 mattrobball
author:mattrobball
mrb/cover data fields --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict 949/657 Mathlib/Algebra/Algebra/Equiv.lean,Mathlib/Algebra/Algebra/Hom.lean,Mathlib/Algebra/Associated.lean,Mathlib/Algebra/Category/MonCat/Colimits.lean,Mathlib/Algebra/Category/Ring/Colimits.lean,Mathlib/Algebra/DirectSum/Ring.lean,Mathlib/Algebra/Field/Basic.lean,Mathlib/Algebra/Field/IsField.lean,Mathlib/Algebra/Free.lean,Mathlib/Algebra/FreeMonoid/Basic.lean,Mathlib/Algebra/GradedMonoid.lean,Mathlib/Algebra/Group/Aut.lean,Mathlib/Algebra/Group/Hom/Defs.lean,Mathlib/Algebra/Group/Hom/Instances.lean,Mathlib/Algebra/Group/InjSurj.lean,Mathlib/Algebra/Group/Opposite.lean,Mathlib/Algebra/Group/Pi/Lemmas.lean,Mathlib/Algebra/Group/TypeTags.lean,Mathlib/Algebra/Group/Units.lean,Mathlib/Algebra/Group/WithOne/Defs.lean,Mathlib/Algebra/GroupWithZero/Basic.lean,Mathlib/Algebra/GroupWithZero/InjSurj.lean,Mathlib/Algebra/Lie/NonUnitalNonAssocAlgebra.lean,Mathlib/Algebra/Module/Basic.lean,Mathlib/Algebra/Module/Equiv.lean,Mathlib/Algebra/Module/LocalizedModule.lean,Mathlib/Algebra/Order/Group/Cone.lean,Mathlib/Algebra/Order/Interval.lean,Mathlib/Algebra/Order/Monoid/WithTop.lean,Mathlib/Algebra/Order/Ring/WithTop.lean,Mathlib/Algebra/PEmptyInstances.lean,Mathlib/Algebra/Quandle.lean,Mathlib/Algebra/Ring/Aut.lean,Mathlib/Algebra/Ring/Defs.lean,Mathlib/Algebra/Ring/Hom/Defs.lean,Mathlib/Algebra/Ring/InjSurj.lean,Mathlib/Algebra/Ring/Opposite.lean,Mathlib/Algebra/Ring/Pi.lean,Mathlib/Algebra/Ring/ULift.lean,Mathlib/Algebra/SMulWithZero.lean,Mathlib/Algebra/Star/StarAlgHom.lean,Mathlib/Algebra/Tropical/Basic.lean,Mathlib/Analysis/Fourier/FourierTransformDeriv.lean,Mathlib/Analysis/NormedSpace/ContinuousAffineMap.lean,Mathlib/Analysis/NormedSpace/HahnBanach/Extension.lean,Mathlib/Analysis/NormedSpace/OperatorNorm/Basic.lean,Mathlib/Analysis/SpecialFunctions/PolarCoord.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Deriv.lean,Mathlib/CategoryTheory/Endomorphism.lean,Mathlib/CategoryTheory/Groupoid/VertexGroup.lean,Mathlib/CategoryTheory/Monoidal/Internal/Module.lean,Mathlib/Combinatorics/Quiver/SingleObj.lean,Mathlib/Combinatorics/Quiver/Symmetric.lean,Mathlib/Combinatorics/Young/YoungDiagram.lean,Mathlib/Control/Applicative.lean,Mathlib/Control/Basic.lean,Mathlib/Control/Functor.lean,Mathlib/Control/Monad/Cont.lean,Mathlib/Control/ULift.lean,Mathlib/Data/Erased.lean,Mathlib/Data/Int/Basic.lean,Mathlib/Data/Int/Cast/Prod.lean,Mathlib/Data/Nat/Basic.lean,Mathlib/Data/Nat/Cast/Defs.lean,Mathlib/Data/Nat/Order/Basic.lean,Mathlib/Data/Num/Lemmas.lean,Mathlib/Data/PSigma/Order.lean,Mathlib/Data/Prod/Lex.lean,Mathlib/Data/Quot.lean,Mathlib/Data/Rat/Defs.lean,Mathlib/Data/Set/Basic.lean,Mathlib/Data/Set/Semiring.lean,Mathlib/Data/Sigma/Order.lean,Mathlib/Data/Sign.lean,Mathlib/Data/Sum/Lattice.lean,Mathlib/Data/Sum/Order.lean,Mathlib/Data/TwoPointing.lean,Mathlib/Data/ZMod/Defs.lean,Mathlib/GroupTheory/FreeGroup/Basic.lean,Mathlib/GroupTheory/GroupAction/Basic.lean,Mathlib/GroupTheory/GroupAction/Defs.lean,Mathlib/GroupTheory/GroupAction/Opposite.lean,Mathlib/GroupTheory/GroupAction/Option.lean,Mathlib/GroupTheory/GroupAction/Prod.lean,Mathlib/GroupTheory/GroupAction/SubMulAction/Pointwise.lean,Mathlib/GroupTheory/GroupAction/Units.lean,Mathlib/GroupTheory/MonoidLocalization.lean,Mathlib/GroupTheory/Perm/Basic.lean,Mathlib/GroupTheory/Subgroup/Basic.lean,Mathlib/GroupTheory/Submonoid/Operations.lean,Mathlib/GroupTheory/Submonoid/Pointwise.lean,Mathlib/GroupTheory/Subsemigroup/Operations.lean,Mathlib/Init/Data/Int/Order.lean,Mathlib/Init/Data/List/Instances.lean,Mathlib/Init/Data/Nat/Lemmas.lean,Mathlib/LinearAlgebra/AffineSpace/AffineMap.lean,Mathlib/LinearAlgebra/Basis.lean,Mathlib/Logic/Nontrivial/Basic.lean,Mathlib/Logic/Unique.lean,Mathlib/MeasureTheory/Integral/Bochner.lean 120 13 ['YaelDillies', 'grunweg', 'leanprover-bot', 'mattrobball'] nobody
54-47388
1 month ago
452-78060
1 year ago
0-0
0 seconds
12673 grunweg
author:grunweg
feat: add ContDiff.lipschitzOnWith A C¹ function is Lipschitz on each convex compact set. From sphere-eversion. -------- Commits can be reviewed independently. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis merge-conflict awaiting-author help-wanted 30/11 Mathlib/Analysis/Calculus/ContDiff/RCLike.lean 1 6 ['Ruben-VandeVelde', 'github-actions', 'grunweg', 'sgouezel'] nobody
53-16899
1 month ago
53-16899
1 month ago
1-7552
1 day
21238 joneugster
author:joneugster
feat(Cache): enable partial cache in downstream projects Add features to `cache` and cleanup code: * enable partial cache retrieval in downstream projects: `lake exe cache get MyProject.Basic` downloads only the relevant cache to build `MyProject/Basic.lean` * accept paths `Mathlib/Init.lean` and modules `Mathlib.Init` likewise #21822 * accept folders in the form `Mathlib/Data` or `Mathlib.Data` and does a directory walk to find all`.lean` files therein #21838 * throw error if sources contain a build loop. #21632 * cleanup * internally cache now works with the module names as keys (used paths before) #21834 * eliminate need of parsing the `lake_manifest.json`, use the Lean search path from `LEAN_SRC_PATH` instead. #21666 * eliminate most hard-coded file paths, generating them from the module name with `Lean.findLean` #21818 * add documentation --- - [x] depends on: #21834 - [ ] depends on: #21838 ### Follow-up PR: - #21842 ### Notes: - replaces: #21195 - should address: #8767 - should address: #20568 ### Completed: - [x] depends on: #21632 - [x] ~~depends on: #21663~~ - [x] depends on: #21666 - [x] depends on: #21701 - [x] depends on: #21703 - [x] depends on: #21704 - [x] depends on: #21705 - [x] depends on: #21707 - [x] depends on: #21711 - [x] depends on: #21750 - [x] depends on: #21815 - [x] depends on: #21816 - [x] depends on: #21817 - [x] depends on: #21818 - [x] depends on: #21822 - [x] depends on: #21830 - #21848 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) CI t-meta merge-conflict blocked-by-other-PR 231/118 Cache/Hashing.lean,Cache/IO.lean,Cache/Main.lean 3 n/a ['github-actions', 'grunweg', 'joneugster', 'kim-em', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
53-4165
1 month ago
unknown
unknown
21842 joneugster
author:joneugster
refactor(Cache): use module name for file hash instead of non-resolved file path This invalidates cache once, similarly to when the `lean-toolchain` gets bumped or the `lakefile` modified. --- - [ ] depends on: #21238 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) CI t-meta merge-conflict blocked-by-other-PR 284/139 Cache/Hashing.lean,Cache/IO.lean,Cache/Lean.lean,Cache/Main.lean 4 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
53-4041
1 month ago
116-1064
3 months ago*
0-0
0 seconds*
19467 quangvdao
author:quangvdao
feat(MvPolynomial/Equiv): Add `MvPolynomial.finSuccEquivNth` This PR adds `MvPolynomial.finSuccEquivNth`, which is the algebra isomorphism between `MvPolynomial (Fin (n + 1)) R` and `Polynomial (MvPolynomial (Fin n) R)` by identifying the `p`-th variable as the indeterminate. This generalizes `MvPolynomial.finSuccEquiv` which is only for the `0`-th variable. The supporting theorems for the `Nth` version are identical to the current version, with the `Nth` version deduced from the former. These changes require new definitions in `Finsupp/Fin`, which is a separate PR. Co-authored-by: Yaël Dillies --- - [ ] depends on: #19315 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict blocked-by-other-PR
label:t-algebra$
541/163 Mathlib/Algebra/BigOperators/Fin.lean,Mathlib/Algebra/BigOperators/Finsupp.lean,Mathlib/Algebra/MvPolynomial/Equiv.lean,Mathlib/Data/Fin/Basic.lean,Mathlib/Data/Fin/Tuple/Basic.lean,Mathlib/Data/Finsupp/Fin.lean,scripts/nolints_prime_decls.txt 7 9 ['acmepjz', 'github-actions', 'grunweg', 'mathlib4-dependent-issues-bot', 'quangvdao'] nobody
52-84662
1 month ago
52-84662
1 month ago
0-790
13 minutes
20567 grunweg
author:grunweg
feat(Cache): two small features - add an informational message to the get command (when run without arguments): when more than 80% of all cache files present were not used in the last command, tell the user about the `clean` command --- - [ ] depends on #20568 (for the first feature) - [ ] TODO: re-design this feature and the clean command: if there are N local copies of mathlib, cache should have a pointer to all of them - to avoid clearing all N-1 from inside the last local copy [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta merge-conflict 38/2 Cache/Main.lean 1 11 ['Julian', 'arthurpaulino', 'fpvandoorn', 'github-actions', 'grunweg'] nobody
52-84649
1 month ago
52-84649
1 month ago
1-17369
1 day
20313 thefundamentaltheor3m
author:thefundamentaltheor3m
feat(Data/Complex/Exponential): prove some useful results about the complex exponential. This PR proves two basic results about the complex exponential: * `abs_exp_mul_I (x : ℂ) : abs (Complex.exp (I * x)) = Real.exp (-x.im)` * `one_sub_rexp_re_le_abs_one_sub_cexp (x : ℂ) : 1 - Real.exp x.re ≤ Complex.abs (1 - Complex.exp x)` Both results were proved as part of the sphere packing project. There's a chance they're too specific for mathlib, but I thought they were worth PRing anyway. Would it also be a good idea to tag `abs_exp_mul_I` with `simp`? Feedback/suggestions welcome. Note: `one_sub_rexp_re_le_abs_one_sub_cexp` was proved by Bhavik Mehta @b-mehta --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-analysis merge-conflict 167/141 Mathlib.lean,Mathlib/Analysis/Complex/Basic.lean,Mathlib/Analysis/SpecialFunctions/Log/ERealExp.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Chebyshev.lean,Mathlib/Data/Complex/Exponential/Defs.lean,Mathlib/Data/Complex/Exponential/Lemmas.lean,Mathlib/Data/Complex/ExponentialBounds.lean,Mathlib/Tactic/FunProp.lean,MathlibTest/Recall.lean,MathlibTest/positivity.lean 10 12 ['b-mehta', 'github-actions', 'kim-em', 'thefundamentaltheor3m', 'trivial1711'] nobody
52-84615
1 month ago
52-84615
1 month ago
25-60481
25 days
22147 smmercuri
author:smmercuri
feat: collections of distinct infinite places contain values that diverge around 1 For a given infinite place $v$ of a field $K$, there is an $a \in K$ such that $v(a) < 1$ while $w(a) > 1$ for all $w \neq v$ --- - [ ] depends on: #22142 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-algebra t-analysis merge-conflict blocked-by-other-PR
label:t-algebra$
511/2 Mathlib/Algebra/Order/AbsoluteValue/Basic.lean,Mathlib/Analysis/AbsoluteValue/Equivalence.lean,Mathlib/Analysis/Normed/Ring/WithAbs.lean,Mathlib/Data/Fin/Basic.lean,Mathlib/Data/Finset/Lattice/Fold.lean,Mathlib/Logic/Pairwise.lean,Mathlib/NumberTheory/NumberField/Embeddings.lean 7 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
52-84501
1 month ago
52-84501
1 month ago
0-1327
22 minutes
22698 Kiolt
author:Kiolt
feat: notation for whisker(Left/Right)Iso From Toric --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) toric t-category-theory merge-conflict 175/113 Mathlib/Algebra/Homology/Monoidal.lean,Mathlib/CategoryTheory/Bicategory/Adjunction/Basic.lean,Mathlib/CategoryTheory/Bicategory/Basic.lean,Mathlib/CategoryTheory/Bicategory/Coherence.lean,Mathlib/CategoryTheory/Bicategory/Extension.lean,Mathlib/CategoryTheory/Bicategory/Functor/Pseudofunctor.lean,Mathlib/CategoryTheory/Bicategory/NaturalTransformation/Strong.lean,Mathlib/CategoryTheory/Bicategory/SingleObj.lean,Mathlib/CategoryTheory/Closed/Functor.lean,Mathlib/CategoryTheory/Closed/Ideal.lean,Mathlib/CategoryTheory/Enriched/FunctorCategory.lean,Mathlib/CategoryTheory/GradedObject/Monoidal.lean,Mathlib/CategoryTheory/Monoidal/Braided/Basic.lean,Mathlib/CategoryTheory/Monoidal/Braided/Reflection.lean,Mathlib/CategoryTheory/Monoidal/Category.lean,Mathlib/CategoryTheory/Monoidal/Center.lean,Mathlib/CategoryTheory/Monoidal/Free/Coherence.lean,Mathlib/CategoryTheory/Monoidal/Preadditive.lean,Mathlib/CategoryTheory/Monoidal/Transport.lean,Mathlib/Tactic/CategoryTheory/BicategoricalComp.lean,Mathlib/Tactic/CategoryTheory/Bicategory/Datatypes.lean,Mathlib/Tactic/CategoryTheory/Bicategory/Normalize.lean,Mathlib/Tactic/CategoryTheory/Bicategory/PureCoherence.lean,Mathlib/Tactic/CategoryTheory/Monoidal/Datatypes.lean,Mathlib/Tactic/CategoryTheory/Monoidal/Normalize.lean,Mathlib/Tactic/CategoryTheory/Monoidal/PureCoherence.lean,Mathlib/Tactic/CategoryTheory/MonoidalComp.lean 27 21 ['Kiolt', 'YaelDillies', 'b-mehta', 'github-actions', 'leanprover-bot'] nobody
52-84444
1 month ago
52-84444
1 month ago
3-36238
3 days
21714 mattrobball
author:mattrobball
test t-order merge-conflict 13/13 Mathlib/Order/Hom/Lattice.lean,lean-toolchain 2 4 ['github-actions', 'leanprover-bot', 'mattrobball'] nobody
52-83293
1 month ago
52-83293
1 month ago
0-0
0 seconds
20224 joelriou
author:joelriou
feat(AlgebraicTopology/ModelCategory): a trick by Joyal In order to construct a model category, we may sometimes have basically proven all the axioms with the exception of the left lifting property of cofibrations with respect to trivial fibrations. A trick by Joyal allows to obtain this lifting property under suitable assumptions, namely that cofibrations are stable under composition and cobase change. --- - [ ] depends on: #20210 - [ ] depends on: #19158 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-category-theory merge-conflict blocked-by-other-PR 587/4 Mathlib.lean,Mathlib/AlgebraicTopology/ModelCategory/Basic.lean,Mathlib/AlgebraicTopology/ModelCategory/Instances.lean,Mathlib/AlgebraicTopology/ModelCategory/JoyalTrick.lean,Mathlib/CategoryTheory/MorphismProperty/WeakFactorizationSystem.lean,docs/references.bib 6 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
52-82507
1 month ago
61-79903
2 months ago
0-15
15 seconds
20781 artie2000
author:artie2000
feat(Algebra): Add Aesop automation around `Even` / `IsSquare`. * Add `aesop` attributes to enable automation for goals of the form `Even x`, `IsSquare x` and `IsSumSq x` * Add test examples * Replace some existing proofs with `by aesop` The automation follows the principles of #20477 -- see library note [SetLike Aesop lemmas]. --- - [x] depends on: #16094 - [ ] depends on: #20818 - [ ] depends on: #20477 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict blocked-by-other-PR
label:t-algebra$
257/117 Mathlib/Algebra/Algebra/NonUnitalSubalgebra.lean,Mathlib/Algebra/Algebra/Subalgebra/Basic.lean,Mathlib/Algebra/Field/Subfield/Basic.lean,Mathlib/Algebra/Field/Subfield/Defs.lean,Mathlib/Algebra/Group/Even.lean,Mathlib/Algebra/Group/Subgroup/Basic.lean,Mathlib/Algebra/Group/Subgroup/Defs.lean,Mathlib/Algebra/Group/Subgroup/Lattice.lean,Mathlib/Algebra/Group/Submonoid/Basic.lean,Mathlib/Algebra/Group/Submonoid/Defs.lean,Mathlib/Algebra/Group/Submonoid/Pointwise.lean,Mathlib/Algebra/Group/Subsemigroup/Basic.lean,Mathlib/Algebra/Group/Subsemigroup/Defs.lean,Mathlib/Algebra/HierarchyDesign.lean,Mathlib/Algebra/Lie/Subalgebra.lean,Mathlib/Algebra/Lie/Submodule.lean,Mathlib/Algebra/Module/Bimodule.lean,Mathlib/Algebra/Module/Submodule/Defs.lean,Mathlib/Algebra/Module/Submodule/Lattice.lean,Mathlib/Algebra/Order/Ring/Cone.lean,Mathlib/Algebra/Order/Star/Basic.lean,Mathlib/Algebra/Ring/Parity.lean,Mathlib/Algebra/Ring/Subring/Basic.lean,Mathlib/Algebra/Ring/Subring/Defs.lean,Mathlib/Algebra/Ring/Subsemiring/Basic.lean,Mathlib/Algebra/Ring/Subsemiring/Defs.lean,Mathlib/Algebra/Ring/SumsOfSquares.lean,Mathlib/Algebra/Star/Basic.lean,Mathlib/Algebra/Star/NonUnitalSubalgebra.lean,Mathlib/Algebra/Star/SelfAdjoint.lean,Mathlib/Algebra/Star/Subalgebra.lean,Mathlib/Analysis/Convex/Cone/Basic.lean,Mathlib/FieldTheory/IntermediateField/Basic.lean,Mathlib/LinearAlgebra/RootSystem/WeylGroup.lean,Mathlib/LinearAlgebra/Span/Defs.lean,Mathlib/NumberTheory/KummerDedekind.lean,Mathlib/NumberTheory/LegendreSymbol/QuadraticChar/Basic.lean,Mathlib/NumberTheory/LegendreSymbol/QuadraticChar/GaussSum.lean,Mathlib/Order/BooleanSubalgebra.lean,Mathlib/RingTheory/Adjoin/Basic.lean,Mathlib/RingTheory/DedekindDomain/Different.lean,Mathlib/RingTheory/EssentialFiniteness.lean,Mathlib/RingTheory/GradedAlgebra/HomogeneousLocalization.lean,Mathlib/RingTheory/NonUnitalSubring/Basic.lean,Mathlib/RingTheory/NonUnitalSubsemiring/Basic.lean,Mathlib/RingTheory/TwoSidedIdeal/Basic.lean,Mathlib/Topology/Algebra/Algebra.lean,Mathlib/Topology/Algebra/NonUnitalAlgebra.lean,Mathlib/Topology/Algebra/NonUnitalStarAlgebra.lean,Mathlib/Topology/Algebra/StarSubalgebra.lean 50 n/a ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
52-80768
1 month ago
unknown
unknown
20730 kuotsanhsu
author:kuotsanhsu
feat(LinearAlgebra/Matrix/SchurTriangulation): prove Schur decomposition/triangulation `Matrix.schur_triangulation` shows that a matrix over an algebraically closed field is unitarily similar to an upper triangular matrix --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra merge-conflict awaiting-author
label:t-algebra$
317/2 Mathlib.lean,Mathlib/LinearAlgebra/Matrix/Block.lean,Mathlib/LinearAlgebra/Matrix/SchurTriangulation.lean,Mathlib/Logic/Equiv/Basic.lean 4 14 ['eric-wieser', 'github-actions', 'kim-em', 'kuotsanhsu'] nobody
52-80747
1 month ago
52-80747
1 month ago
13-60072
13 days
22754 Parcly-Taxel
author:Parcly-Taxel
chore: clear more `docBlame` nolints --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import tech debt merge-conflict awaiting-author documentation 78/64 Mathlib/Algebra/CharP/MixedCharZero.lean,Mathlib/Algebra/ContinuedFractions/Computation/Basic.lean,Mathlib/Algebra/EuclideanDomain/Defs.lean,Mathlib/Algebra/Module/Injective.lean,Mathlib/Algebra/Notation/Defs.lean,Mathlib/Algebra/Polynomial/Basic.lean,Mathlib/Analysis/BoxIntegral/Partition/Filter.lean,Mathlib/Data/Analysis/Topology.lean,Mathlib/Data/Stream/Defs.lean,Mathlib/Data/Stream/Init.lean,Mathlib/Geometry/RingedSpace/PresheafedSpace.lean,Mathlib/LinearAlgebra/AffineSpace/AffineEquiv.lean,Mathlib/LinearAlgebra/AffineSpace/AffineMap.lean,Mathlib/LinearAlgebra/AffineSpace/Basis.lean,Mathlib/LinearAlgebra/AffineSpace/Independent.lean,Mathlib/LinearAlgebra/Matrix/Transvection.lean,Mathlib/LinearAlgebra/QuadraticForm/Basic.lean,Mathlib/Logic/Equiv/Defs.lean,Mathlib/NumberTheory/ModularForms/SlashActions.lean,Mathlib/NumberTheory/ModularForms/SlashInvariantForms.lean,Mathlib/Order/Atoms.lean,Mathlib/Order/PrimeIdeal.lean,Mathlib/RingTheory/GradedAlgebra/HomogeneousLocalization.lean,Mathlib/RingTheory/PowerBasis.lean,Mathlib/RingTheory/WittVector/Isocrystal.lean,Mathlib/Topology/MetricSpace/GromovHausdorff.lean,Mathlib/Topology/Order/Hom/Esakia.lean,scripts/nolints.json 28 9 ['Parcly-Taxel', 'github-actions', 'jcommelin', 'leanprover-community-bot-assistant'] nobody
52-5824
1 month ago
52-5826
1 month ago
0-3406
56 minutes
19117 eric-wieser
author:eric-wieser
feat: derivatives of matrix operations These are finally possible to state after #19108. However, a lot of bundled `ContinuousLinearMap`s are missing. --- - [x] depends on: #19108 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis merge-conflict WIP 336/22 Mathlib.lean,Mathlib/Analysis/Calculus/Deriv/Matrix.lean,Mathlib/Analysis/Calculus/FDeriv/Basic.lean,Mathlib/Analysis/Calculus/FDeriv/Matrix.lean 4 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
51-16725
1 month ago
51-16727
1 month ago
0-0
0 seconds
12605 FR-vdash-bot
author:FR-vdash-bot
chore: attribute [induction_eliminator] Add attribute [induction_eliminator] to `AdjoinRoot.induction_on` `ENat.recTopCoe` `ENNReal.recTopCoe` `Finset.induction` `Magma.AssocQuotient.induction_on` `ManyOneDegree.ind_on` `Module.Ray.ind` (and add `Orientation.ind` for `Orientation`, an abbrev of it. I wish that we do not need to add it in the future.) `Multiset.induction` `MvPolynomial.induction_on` `OnePoint.rec` `Opposite.rec'` `Ordinal.limitRecOn` `PartENat.casesOn` `Polynomial.induction_on'` `QuotientAddGroup.induction_on'` (and add `AddCircle.induction_on` for `AddCircle`, an abbrev of it. I wish that we do not need to add it in the future.) `QuotientGroup.induction_on'` (doesn't actually work) `Real.Angle.induction_on` `SimplexCategory.rec` `Trunc.induction_on` --- - [x] depends on: #13476 - [x] depends on: #13264 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author 354/342 Mathlib/Algebra/BigOperators/Associated.lean,Mathlib/Algebra/BigOperators/Group/Finset.lean,Mathlib/Algebra/BigOperators/Group/Multiset.lean,Mathlib/Algebra/BigOperators/Ring.lean,Mathlib/Algebra/GCDMonoid/Finset.lean,Mathlib/Algebra/GCDMonoid/Multiset.lean,Mathlib/Algebra/Group/Subgroup/Finite.lean,Mathlib/Algebra/GroupWithZero/WithZero.lean,Mathlib/Algebra/Lie/Submodule.lean,Mathlib/Algebra/Lie/Weights/Basic.lean,Mathlib/Algebra/Module/BigOperators.lean,Mathlib/Algebra/MvPolynomial/Basic.lean,Mathlib/Algebra/MvPolynomial/Derivation.lean,Mathlib/Algebra/MvPolynomial/Variables.lean,Mathlib/Algebra/Order/ToIntervalMod.lean,Mathlib/Algebra/Polynomial/BigOperators.lean,Mathlib/Algebra/Polynomial/Degree/Lemmas.lean,Mathlib/Algebra/Polynomial/Derivative.lean,Mathlib/Algebra/Polynomial/Eval.lean,Mathlib/Algebra/Polynomial/Induction.lean,Mathlib/Algebra/Polynomial/Module/Basic.lean,Mathlib/Algebra/Polynomial/PartialFractions.lean,Mathlib/Algebra/Polynomial/Smeval.lean,Mathlib/Algebra/Tropical/BigOperators.lean,Mathlib/AlgebraicTopology/DoldKan/NCompGamma.lean,Mathlib/AlgebraicTopology/SimplexCategory.lean,Mathlib/AlgebraicTopology/SplitSimplicialObject.lean,Mathlib/Analysis/Analytic/Constructions.lean,Mathlib/Analysis/Asymptotics/Asymptotics.lean,Mathlib/Analysis/BoxIntegral/Basic.lean,Mathlib/Analysis/BoxIntegral/Partition/Additive.lean,Mathlib/Analysis/BoxIntegral/Partition/Split.lean,Mathlib/Analysis/Calculus/ContDiff/Basic.lean,Mathlib/Analysis/Calculus/ContDiff/Bounds.lean,Mathlib/Analysis/Calculus/Deriv/Polynomial.lean,Mathlib/Analysis/Convex/Combination.lean,Mathlib/Analysis/Convex/Exposed.lean,Mathlib/Analysis/Fourier/AddCircle.lean,Mathlib/Analysis/NormedSpace/Exponential.lean,Mathlib/Analysis/NormedSpace/Multilinear/Basic.lean,Mathlib/Analysis/SpecialFunctions/Complex/Arg.lean,Mathlib/Analysis/SpecialFunctions/Complex/Circle.lean,Mathlib/Analysis/SpecialFunctions/Log/Base.lean,Mathlib/Analysis/SpecialFunctions/PolynomialExp.lean,Mathlib/Analysis/SpecialFunctions/Pow/NNReal.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Angle.lean,Mathlib/CategoryTheory/Filtered/Basic.lean,Mathlib/CategoryTheory/Subobject/Lattice.lean,Mathlib/Combinatorics/Additive/PluenneckeRuzsa.lean,Mathlib/Combinatorics/SetFamily/Compression/Down.lean,Mathlib/Combinatorics/SetFamily/FourFunctions.lean,Mathlib/Combinatorics/SetFamily/HarrisKleitman.lean,Mathlib/Computability/Reduce.lean,Mathlib/Data/DFinsupp/Basic.lean,Mathlib/Data/DFinsupp/WellFounded.lean,Mathlib/Data/Finset/Basic.lean,Mathlib/Data/Finset/Fold.lean,Mathlib/Data/Finset/Lattice.lean,Mathlib/Data/Finset/NAry.lean,Mathlib/Data/Fintype/Sum.lean,Mathlib/Data/Multiset/Antidiagonal.lean,Mathlib/Data/Multiset/Basic.lean,Mathlib/Data/Multiset/Bind.lean,Mathlib/Data/Multiset/Fold.lean,Mathlib/Data/Multiset/Lattice.lean,Mathlib/Data/Multiset/Pi.lean,Mathlib/Data/Multiset/Powerset.lean,Mathlib/Data/Multiset/Sections.lean,Mathlib/Data/Nat/Choose/Multinomial.lean,Mathlib/Data/Nat/PartENat.lean,Mathlib/Data/Quot.lean,Mathlib/Data/Set/Pointwise/BigOperators.lean,Mathlib/FieldTheory/IntermediateField.lean,Mathlib/FieldTheory/IsAlgClosed/AlgebraicClosure.lean,Mathlib/Geometry/Manifold/Algebra/Monoid.lean,Mathlib/Geometry/RingedSpace/Basic.lean,Mathlib/Geometry/RingedSpace/OpenImmersion.lean,Mathlib/Geometry/RingedSpace/PresheafedSpace/Gluing.lean,Mathlib/GroupTheory/Coset.lean,Mathlib/GroupTheory/NoncommPiCoprod.lean,Mathlib/GroupTheory/Perm/Cycle/Type.lean,Mathlib/LinearAlgebra/Determinant.lean,Mathlib/LinearAlgebra/Eigenspace/Basic.lean,Mathlib/LinearAlgebra/FiniteDimensional.lean,Mathlib/LinearAlgebra/LinearIndependent.lean,Mathlib/LinearAlgebra/Matrix/Determinant/Basic.lean,Mathlib/LinearAlgebra/Multilinear/Basic.lean,Mathlib/LinearAlgebra/Orientation.lean,Mathlib/LinearAlgebra/Projectivization/Basic.lean,Mathlib/LinearAlgebra/Ray.lean,Mathlib/LinearAlgebra/TensorProduct/Basic.lean,Mathlib/Logic/Hydra.lean,Mathlib/MeasureTheory/Function/ConditionalExpectation/Basic.lean,Mathlib/MeasureTheory/Function/L1Space.lean,Mathlib/MeasureTheory/Function/SimpleFunc.lean,Mathlib/MeasureTheory/Integral/Lebesgue.lean,Mathlib/MeasureTheory/Integral/Marginal.lean,Mathlib/MeasureTheory/Integral/MeanInequalities.lean,Mathlib/MeasureTheory/Integral/SetIntegral.lean,Mathlib/MeasureTheory/Measure/AddContent.lean 140 14 ['FR-vdash-bot', 'YaelDillies', 'eric-wieser', 'github-actions', 'leanprover-community-mathlib4-bot', 'urkud'] nobody
51-11340
1 month ago
337-25266
11 months ago
4-46495
4 days
23916 Vierkantor
author:Vierkantor
chore: upstream shake from Mathlib to Batteries This is an adaptation PR for the upstreaming of shake to Batteries. Zulip discussion: https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Spinning.20off.20.60mathlib-linters.60.20and.20.60shake.60.20repo --- - [ ] depends on: https://github.com/leanprover-community/batteries/pull/1204 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-linter blocked-by-batt-PR merge-conflict blocked-by-other-PR 3/614 Shake/Main.lean,lake-manifest.json,lakefile.lean 3 5 ['Vierkantor', 'github-actions', 'grunweg', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
49-14973
1 month ago
49-14975
1 month ago
0-894
14 minutes
15099 joelriou
author:joelriou
feat(CategoryTheory/Sites): the Mayer-Vietoris long exact sequence in sheaf cohomology In this PR, we obtain the long exact Mayer-Vietoris sequence in sheaf cohomology `... ⟶ H^n₀(S.X₄, F) ⟶ H^n₀(S.X₂, F) ⊞ H^n₀(S.X₃, F) ⟶ H^n₀(S.X₁, F) ⟶ H^n₁(S.X₄, F) ⟶ ...` when `n₀ + 1 = n₁`. It is attached to any "Mayer-Vietoris square", which includes the typical case of a covering by two open subsets in a topological space. (This API shall also apply to the case of Nisnevich distinguished squares of schemes.) --- - [x] depends on: #15770 - [x] depends on: #14793 - [x] depends on: #14515 - [x] depends on: #15092 - [x] depends on: #15053 - [x] depends on: #14867 - [x] depends on: #14959 - [x] depends on: #14957 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory merge-conflict WIP 348/4 Mathlib.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/Basic.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/Biprod.lean,Mathlib/CategoryTheory/Preadditive/Opposite.lean,Mathlib/CategoryTheory/Shift/Basic.lean,Mathlib/CategoryTheory/Shift/ShiftedHom.lean,Mathlib/CategoryTheory/Sites/SheafCohomology/Basic.lean,Mathlib/CategoryTheory/Sites/SheafCohomology/MayerVietoris.lean 8 n/a ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
48-41187
1 month ago
unknown
unknown
23859 urkud
author:urkud
feat(Topology/../Order/Field): generalize to `Semifield` .. from a linear ordered field to a linear ordered semifield--- - [ ] depends on: #23857 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology merge-conflict 245/219 Mathlib/Algebra/Order/Group/Pointwise/Interval.lean,Mathlib/Analysis/BoxIntegral/Box/SubboxInduction.lean,Mathlib/Topology/Algebra/Order/Field.lean,Mathlib/Topology/Order/Basic.lean 4 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
48-37163
1 month ago
48-37166
1 month ago
0-265
4 minutes
22782 alreadydone
author:alreadydone
WIP: etale space associated to a presheaf --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology merge-conflict WIP 349/170 Mathlib.lean,Mathlib/CategoryTheory/Category/Pairwise.lean,Mathlib/Topology/EtaleSpace.lean,Mathlib/Topology/Sheaves/LocalPredicate.lean,Mathlib/Topology/Sheaves/PresheafOfFunctions.lean,Mathlib/Topology/Sheaves/SheafCondition/OpensLeCover.lean,Mathlib/Topology/Sheaves/SheafCondition/PairwiseIntersections.lean,Mathlib/Topology/Sheaves/SheafCondition/UniqueGluing.lean,Mathlib/Topology/Sheaves/SheafOfFunctions.lean,Mathlib/Topology/Sheaves/Sheafify.lean,Mathlib/Topology/Sheaves/Stalks.lean 11 2 ['github-actions', 'leanprover-community-bot-assistant'] nobody
48-29614
1 month ago
48-29616
1 month ago
0-687
11 minutes
22908 AntoineChambert-Loir
author:AntoineChambert-Loir
feat(RingTheory/Finiteness/Small): tensor product of the system of small submodules The directed limit of a tensor product for the directed system of small submodules. Co-authored with @mariainesdff --- - [ ] depends on: #22898 - [x] depends on: #22911 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict blocked-by-other-PR
label:t-algebra$
624/2 Mathlib.lean,Mathlib/RingTheory/Adjoin/FG.lean,Mathlib/RingTheory/Finiteness/Basic.lean,Mathlib/RingTheory/Finiteness/Cardinality.lean,Mathlib/RingTheory/Finiteness/Small.lean,Mathlib/RingTheory/Spectrum/Prime/RingHom.lean,Mathlib/RingTheory/TensorProduct/Basic.lean,Mathlib/RingTheory/TensorProduct/DirectLimit/FG.lean,Mathlib/RingTheory/TensorProduct/DirectLimit/Small.lean 9 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
47-80875
1 month ago
74-15438
2 months ago
0-3552
59 minutes
21696 bryangingechen
author:bryangingechen
generalize toAdditive frontend to allow use of other translations TODO (maybe split off into future PRs?): - further extract to_additive specific stuff - rename functions - update docstrings - write a PR description --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta merge-conflict 229/174 Mathlib/GroupTheory/Coset/Defs.lean,Mathlib/Tactic/ToAdditive/Frontend.lean,MathlibTest/toAdditive.lean 3 2 ['github-actions', 'leanprover-community-bot-assistant'] nobody
47-40689
1 month ago
47-40691
1 month ago
0-0
0 seconds
18893 vihdzp
author:vihdzp
feat(Order/InitialSeg): `InitialSeg.exists_relIso_sum` If `r` is an initial segment of `s`, there exists some other relation `t` with `Sum.Lex r t ≃r s`. --- - [x] depends on: #17989 - [ ] depends on: #20409 The names `sumLexLtLE` and `sumLexLeLT` are very sketch, and better suggestions are welcome. Likewise it'd be cool if anyone can figure out how to golf these results. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order merge-conflict awaiting-author blocked-by-other-PR 102/10 Mathlib/Order/InitialSeg.lean,Mathlib/Order/RelIso/Basic.lean,Mathlib/Order/RelIso/Set.lean,Mathlib/SetTheory/Ordinal/Basic.lean 4 13 ['YaelDillies', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'vihdzp'] nobody
47-25576
1 month ago
47-25578
1 month ago
46-65043
46 days
23810 b-reinke
author:b-reinke
chore(Order/Interval): generalize succ/pred lemmas to partial orders Many lemmas in `Mathlib/Order/Interval/Set/SuccPred.lean`and `Mathlib/Order/Interval/Finset/SuccPred.lean` also work for partial orders. They are generalized in this PR by introducing different sections for `PartialOrder` and `LinearOrder` assumptions in the respective files. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order merge-conflict 231/89 Mathlib/Order/Interval/Finset/SuccPred.lean,Mathlib/Order/Interval/Set/SuccPred.lean 2 2 ['github-actions', 'leanprover-community-bot-assistant'] nobody
46-13938
1 month ago
46-13940
1 month ago
16-29623
16 days
24285 madvorak
author:madvorak
chore(Algebra/*-{Category,Homology}): remove unnecessary universe variables Discussions: https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Call.20for.20help.3A.20technical.2F.20organisational.20debt/with/513620128 https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Algebra.20and.20.60Type*.60/with/513558902 https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Task.2026.3A.20Replace.20Type.20u.20by.20Type*.20wherever.20possible/with/513592993 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict
label:t-algebra$
542/916 Mathlib/Algebra/AddTorsor/Basic.lean,Mathlib/Algebra/Algebra/Defs.lean,Mathlib/Algebra/Algebra/Equiv.lean,Mathlib/Algebra/Algebra/Field.lean,Mathlib/Algebra/Algebra/Hom.lean,Mathlib/Algebra/Algebra/Operations.lean,Mathlib/Algebra/Algebra/Spectrum/Basic.lean,Mathlib/Algebra/Algebra/Subalgebra/Lattice.lean,Mathlib/Algebra/Algebra/Subalgebra/Tower.lean,Mathlib/Algebra/Algebra/Tower.lean,Mathlib/Algebra/Central/Basic.lean,Mathlib/Algebra/Central/Defs.lean,Mathlib/Algebra/Central/TensorProduct.lean,Mathlib/Algebra/CharP/Pi.lean,Mathlib/Algebra/CharP/Quotient.lean,Mathlib/Algebra/CharP/Subring.lean,Mathlib/Algebra/DirectSum/Algebra.lean,Mathlib/Algebra/DirectSum/Basic.lean,Mathlib/Algebra/DirectSum/Finsupp.lean,Mathlib/Algebra/DirectSum/Module.lean,Mathlib/Algebra/EuclideanDomain/Basic.lean,Mathlib/Algebra/EuclideanDomain/Defs.lean,Mathlib/Algebra/Field/Basic.lean,Mathlib/Algebra/Field/Defs.lean,Mathlib/Algebra/Field/IsField.lean,Mathlib/Algebra/Field/MinimalAxioms.lean,Mathlib/Algebra/Field/Subfield/Basic.lean,Mathlib/Algebra/Field/Subfield/Defs.lean,Mathlib/Algebra/FreeNonUnitalNonAssocAlgebra.lean,Mathlib/Algebra/Group/Conj.lean,Mathlib/Algebra/Group/Defs.lean,Mathlib/Algebra/Group/Equiv/Finite.lean,Mathlib/Algebra/Group/Ext.lean,Mathlib/Algebra/Group/Hom/End.lean,Mathlib/Algebra/Group/Hom/Instances.lean,Mathlib/Algebra/Group/Invertible/Basic.lean,Mathlib/Algebra/Group/Invertible/Defs.lean,Mathlib/Algebra/Group/Pi/Basic.lean,Mathlib/Algebra/Group/Pi/Lemmas.lean,Mathlib/Algebra/Group/TypeTags/Basic.lean,Mathlib/Algebra/Group/TypeTags/Finite.lean,Mathlib/Algebra/Group/TypeTags/Hom.lean,Mathlib/Algebra/Group/Units/Basic.lean,Mathlib/Algebra/Group/Units/Defs.lean,Mathlib/Algebra/Group/Units/Hom.lean,Mathlib/Algebra/Group/WithOne/Basic.lean,Mathlib/Algebra/Group/WithOne/Defs.lean,Mathlib/Algebra/GroupWithZero/Action/Pi.lean,Mathlib/Algebra/GroupWithZero/Defs.lean,Mathlib/Algebra/GroupWithZero/Invertible.lean,Mathlib/Algebra/GroupWithZero/NeZero.lean,Mathlib/Algebra/Lie/Abelian.lean,Mathlib/Algebra/Lie/Basic.lean,Mathlib/Algebra/Lie/CartanMatrix.lean,Mathlib/Algebra/Lie/CartanSubalgebra.lean,Mathlib/Algebra/Lie/Character.lean,Mathlib/Algebra/Lie/Classical.lean,Mathlib/Algebra/Lie/DirectSum.lean,Mathlib/Algebra/Lie/Free.lean,Mathlib/Algebra/Lie/Ideal.lean,Mathlib/Algebra/Lie/IdealOperations.lean,Mathlib/Algebra/Lie/Matrix.lean,Mathlib/Algebra/Lie/Nilpotent.lean,Mathlib/Algebra/Lie/NonUnitalNonAssocAlgebra.lean,Mathlib/Algebra/Lie/OfAssociative.lean,Mathlib/Algebra/Lie/Quotient.lean,Mathlib/Algebra/Lie/SkewAdjoint.lean,Mathlib/Algebra/Lie/Solvable.lean,Mathlib/Algebra/Lie/Subalgebra.lean,Mathlib/Algebra/Lie/Submodule.lean,Mathlib/Algebra/Lie/TensorProduct.lean,Mathlib/Algebra/Lie/UniversalEnveloping.lean,Mathlib/Algebra/Module/Basic.lean,Mathlib/Algebra/Module/CharacterModule.lean,Mathlib/Algebra/Module/DedekindDomain.lean,Mathlib/Algebra/Module/Defs.lean,Mathlib/Algebra/Module/End.lean,Mathlib/Algebra/Module/Equiv/Opposite.lean,Mathlib/Algebra/Module/Lattice.lean,Mathlib/Algebra/Module/LinearMap/Basic.lean,Mathlib/Algebra/Module/LinearMap/Defs.lean,Mathlib/Algebra/Module/LinearMap/End.lean,Mathlib/Algebra/Module/LocalizedModule/Basic.lean,Mathlib/Algebra/Module/MinimalAxioms.lean,Mathlib/Algebra/Module/NatInt.lean,Mathlib/Algebra/Module/Opposite.lean,Mathlib/Algebra/Module/Pi.lean,Mathlib/Algebra/Module/Presentation/Differentials.lean,Mathlib/Algebra/Module/Presentation/Tensor.lean,Mathlib/Algebra/Module/Rat.lean,Mathlib/Algebra/Module/RingHom.lean,Mathlib/Algebra/Module/Submodule/Basic.lean,Mathlib/Algebra/Module/Torsion.lean,Mathlib/Algebra/MonoidAlgebra/Basic.lean,Mathlib/Algebra/MonoidAlgebra/Defs.lean,Mathlib/Algebra/MonoidAlgebra/Support.lean,Mathlib/Algebra/MvPolynomial/Basic.lean,Mathlib/Algebra/MvPolynomial/CommRing.lean,Mathlib/Algebra/MvPolynomial/Degrees.lean,Mathlib/Algebra/MvPolynomial/Equiv.lean 182 22 ['erdOne', 'github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'madvorak', 'mattrobball'] nobody
46-2635
1 month ago
46-2636
1 month ago
2-12022
2 days
8370 eric-wieser
author:eric-wieser
refactor(Analysis/NormedSpace/Exponential): remove the `𝕂` argument from `exp` This argument is still needed for almost all the lemmas, which means it can longer be found by unification. We keep around `expSeries 𝕂 A`, as it's needed for talking about the radius of convergence over different base fields. This is a prerequisite for #8372, as we can't merge the functions until they have the same interface.\ Zulip thread: [#mathlib4 > Real.exp @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Real.2Eexp/near/401602245) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) This is started from the mathport output on https://github.com/leanprover-community/mathlib/pull/19244 awaiting-zulip t-analysis merge-conflict 432/387 Mathlib/Analysis/CStarAlgebra/Exponential.lean,Mathlib/Analysis/CStarAlgebra/Spectrum.lean,Mathlib/Analysis/Normed/Algebra/Exponential.lean,Mathlib/Analysis/Normed/Algebra/MatrixExponential.lean,Mathlib/Analysis/Normed/Algebra/QuaternionExponential.lean,Mathlib/Analysis/Normed/Algebra/Spectrum.lean,Mathlib/Analysis/Normed/Algebra/TrivSqZeroExt.lean,Mathlib/Analysis/NormedSpace/DualNumber.lean,Mathlib/Analysis/SpecialFunctions/ContinuousFunctionalCalculus/ExpLog.lean,Mathlib/Analysis/SpecialFunctions/Exponential.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Series.lean 11 29 ['YaelDillies', 'eric-wieser', 'girving', 'github-actions', 'j-loreaux', 'kbuzzard', 'leanprover-community-bot-assistant', 'urkud'] nobody
45-69965
1 month ago
57-12195
1 month ago
29-60989
29 days
23621 FR-vdash-bot
author:FR-vdash-bot
chore: deprecate `LinearOrderedComm{Monoid, Group}WithZero` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) - [x] depends on: #20676 t-order t-algebra merge-conflict
label:t-algebra$
261/205 Archive/Imo/Imo1998Q2.lean,Counterexamples/LinearOrderWithPosMulPosEqZero.lean,Mathlib/Algebra/Order/Field/Canonical.lean,Mathlib/Algebra/Order/Field/Rat.lean,Mathlib/Algebra/Order/Floor/Ring.lean,Mathlib/Algebra/Order/GroupWithZero/Canonical.lean,Mathlib/Algebra/Order/GroupWithZero/Finset.lean,Mathlib/Algebra/Order/Hom/Monoid.lean,Mathlib/Algebra/Order/Nonneg/Field.lean,Mathlib/Algebra/Order/Nonneg/Ring.lean,Mathlib/Algebra/Order/Ring/Nat.lean,Mathlib/Combinatorics/Additive/PluenneckeRuzsa.lean,Mathlib/Combinatorics/SimpleGraph/Triangle/Basic.lean,Mathlib/Data/ENNReal/Basic.lean,Mathlib/Data/NNRat/Lemmas.lean,Mathlib/Data/NNReal/Defs.lean,Mathlib/Data/Rat/Cast/Order.lean,Mathlib/FieldTheory/IntermediateField/Adjoin/Defs.lean,Mathlib/FieldTheory/RatFunc/AsPolynomial.lean,Mathlib/GroupTheory/ArchimedeanDensely.lean,Mathlib/NumberTheory/EllipticDivisibilitySequence.lean,Mathlib/NumberTheory/FunctionField.lean,Mathlib/NumberTheory/Ostrowski.lean,Mathlib/RingTheory/Valuation/Archimedean.lean,Mathlib/RingTheory/Valuation/Basic.lean,Mathlib/RingTheory/Valuation/ExtendToLocalization.lean,Mathlib/RingTheory/Valuation/Integers.lean,Mathlib/RingTheory/Valuation/Integral.lean,Mathlib/RingTheory/Valuation/Minpoly.lean,Mathlib/RingTheory/Valuation/Quotient.lean,Mathlib/RingTheory/Valuation/RankOne.lean,Mathlib/RingTheory/Valuation/ValExtension.lean,Mathlib/RingTheory/Valuation/ValuationRing.lean,Mathlib/RingTheory/Valuation/ValuationSubring.lean,Mathlib/SetTheory/Cardinal/Order.lean,Mathlib/Topology/Algebra/Valued/LocallyCompact.lean,Mathlib/Topology/Algebra/Valued/NormedValued.lean,Mathlib/Topology/Algebra/Valued/ValuationTopology.lean,Mathlib/Topology/Algebra/Valued/ValuedField.lean,Mathlib/Topology/Algebra/Valued/WithVal.lean,Mathlib/Topology/Algebra/WithZeroTopology.lean,Mathlib/Topology/UnitInterval.lean,MathlibTest/instance_diamonds.lean,scripts/noshake.json 44 n/a ['FR-vdash-bot', 'github-actions', 'grunweg', 'leanprover-bot', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] kbuzzard
assignee:kbuzzard
45-2205
1 month ago
unknown
unknown
14931 eric-wieser
author:eric-wieser
feat: volume of a simplex --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-euclidean-geometry merge-conflict 207/0 Mathlib/Geometry/Euclidean/Basic.lean,Mathlib/Geometry/Euclidean/Circumcenter.lean,Mathlib/Geometry/Euclidean/Volume.lean 3 3 ['eric-wieser', 'github-actions', 'leanprover-community-bot-assistant'] nobody
44-15092
1 month ago
44-15094
1 month ago
0-0
0 seconds
22583 imathwy
author:imathwy
feat: affinespace homeomorphism There exists a homeomorphism (a continuous bijection with a continuous inverse) between an affine subspace s of a vector space V over a field 𝕜 and its direction s.direction , given a chosen point z ∈ s . --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict awaiting-author
label:t-algebra$
64/2 Mathlib/Analysis/Normed/Group/AddTorsor.lean,Mathlib/LinearAlgebra/AffineSpace/ContinuousAffineEquiv.lean,Mathlib/Topology/Algebra/ConstMulAction.lean,Mathlib/Topology/Algebra/MulAction.lean 4 6 ['JovanGerb', 'eric-wieser', 'github-actions', 'grunweg'] nobody
44-12810
1 month ago
84-57903
2 months ago
0-18122
5 hours
21719 bryangingechen
author:bryangingechen
to_dual attribute Builds on #21696: https://github.com/leanprover-community/mathlib4/compare/bgc-to-additive-0...bgc-order-dual-scratch-0 TODO: - `WithBot.le` -> `WithTop.le` is broken in `WithBot.lean`: I think I understand this now. I need to reorder the arguments of one of the fields of the instance, but it looks like the tactic doesn't support this - naming probably gets screwed up --- - [ ] depends on: #21696 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-meta merge-conflict blocked-by-other-PR 1219/491 Mathlib/CategoryTheory/Category/Basic.lean,Mathlib/CategoryTheory/Functor/Basic.lean,Mathlib/CategoryTheory/Iso.lean,Mathlib/CategoryTheory/NatTrans.lean,Mathlib/Combinatorics/Quiver/Basic.lean,Mathlib/Combinatorics/Quiver/Prefunctor.lean,Mathlib/GroupTheory/Coset/Defs.lean,Mathlib/Lean/Expr/ReplaceRec.lean,Mathlib/Order/Basic.lean,Mathlib/Order/Defs/LinearOrder.lean,Mathlib/Order/Defs/PartialOrder.lean,Mathlib/Order/Notation.lean,Mathlib/Order/OrdContinuous.lean,Mathlib/Order/TypeTags.lean,Mathlib/Order/WithBot.lean,Mathlib/Tactic/CategoryTheory/Reassoc.lean,Mathlib/Tactic/ToAdditive/Frontend.lean,MathlibTest/orderDual.lean,MathlibTest/toAdditive.lean 19 5 ['JovanGerb', 'bryangingechen', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
43-65088
1 month ago
47-40690
1 month ago
0-0
0 seconds
24243 Timeroot
author:Timeroot
feat(Analysis/Calculus/FDeriv): Fderiv on torsors Experiment to see how this goes for now, see [Zulip discussion](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Upgrade.20.60fderiv.60.20to.20.60AddTorsor.60) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis merge-conflict 539/447 Mathlib/Algebra/AddTorsor/Defs.lean,Mathlib/Analysis/Calculus/Deriv/Basic.lean,Mathlib/Analysis/Calculus/Deriv/Prod.lean,Mathlib/Analysis/Calculus/Deriv/Slope.lean,Mathlib/Analysis/Calculus/FDeriv/Add.lean,Mathlib/Analysis/Calculus/FDeriv/Basic.lean,Mathlib/Analysis/Calculus/FDeriv/Bilinear.lean,Mathlib/Analysis/Calculus/FDeriv/Equiv.lean,Mathlib/Analysis/Calculus/FDeriv/Linear.lean,Mathlib/Analysis/Calculus/FDeriv/Measurable.lean,Mathlib/Analysis/Calculus/FDeriv/Mul.lean,Mathlib/Analysis/Calculus/FDeriv/Symmetric.lean,Mathlib/Analysis/Calculus/Gradient/Basic.lean,Mathlib/Analysis/Calculus/LineDeriv/Basic.lean,Mathlib/Analysis/Calculus/LocalExtr/Basic.lean,Mathlib/Analysis/Calculus/ParametricIntegral.lean,Mathlib/Analysis/Calculus/Rademacher.lean,Mathlib/Analysis/Calculus/TangentCone.lean,Mathlib/Analysis/Calculus/UniformLimitsDeriv.lean,Mathlib/Analysis/Complex/Periodic.lean,Mathlib/Analysis/Complex/RealDeriv.lean,Mathlib/Analysis/MellinTransform.lean,Mathlib/Analysis/Normed/Group/Uniform.lean,Mathlib/Analysis/Normed/Module/Basic.lean,Mathlib/Analysis/SpecialFunctions/ExpDeriv.lean,Mathlib/Analysis/SpecialFunctions/Exponential.lean,Mathlib/Analysis/SpecialFunctions/Gamma/Deriv.lean,Mathlib/Analysis/SpecialFunctions/Pow/Deriv.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/EulerSineProd.lean,Mathlib/Geometry/Manifold/IntegralCurve/Transform.lean,Mathlib/Geometry/Manifold/IsManifold/Basic.lean,Mathlib/Geometry/Manifold/MFDeriv/Basic.lean,Mathlib/Geometry/Manifold/MFDeriv/SpecificFunctions.lean,Mathlib/NumberTheory/EulerProduct/ExpLog.lean,Mathlib/NumberTheory/Harmonic/GammaDeriv.lean,Mathlib/NumberTheory/LSeries/Nonvanishing.lean,MathlibTest/Recall.lean 37 3 ['github-actions', 'leanprover-community-bot-assistant'] nobody
42-82348
1 month ago
42-82349
1 month ago
0-0
0 seconds
24322 mattrobball
author:mattrobball
chore: merge repeated `Type*` binders Per the discussion on [Zulip](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Task.2026.3A.20Replace.20Type.20u.20by.20Type*.20wherever.20possible), this PR merges `(A : Type*) (B : Type u)` into `(A B : Type*)` and similarly for `{}`. NOTE: the Python script used it currently in the `/scripts` folder. It is there for inspection and should be removed before merging this PR. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author 685/591 Archive/Imo/Imo2019Q2.lean,Archive/Wiedijk100Theorems/HeronsFormula.lean,Mathlib/Algebra/AddTorsor/Basic.lean,Mathlib/Algebra/AddTorsor/Defs.lean,Mathlib/Algebra/Algebra/Basic.lean,Mathlib/Algebra/Algebra/Pi.lean,Mathlib/Algebra/Algebra/Subalgebra/Pointwise.lean,Mathlib/Algebra/Algebra/Unitization.lean,Mathlib/Algebra/BigOperators/Fin.lean,Mathlib/Algebra/BigOperators/Finsupp/Basic.lean,Mathlib/Algebra/Category/ModuleCat/ChangeOfRings.lean,Mathlib/Algebra/DirectSum/Internal.lean,Mathlib/Algebra/FreeMonoid/Basic.lean,Mathlib/Algebra/Group/Action/Defs.lean,Mathlib/Algebra/Group/Action/Faithful.lean,Mathlib/Algebra/Group/Action/Sigma.lean,Mathlib/Algebra/Group/Hom/Basic.lean,Mathlib/Algebra/Group/Hom/Defs.lean,Mathlib/Algebra/Group/InjSurj.lean,Mathlib/Algebra/Group/Invertible/Basic.lean,Mathlib/Algebra/Group/Prod.lean,Mathlib/Algebra/Group/Subgroup/Basic.lean,Mathlib/Algebra/Group/Subgroup/Ker.lean,Mathlib/Algebra/Group/Submonoid/Basic.lean,Mathlib/Algebra/Group/Submonoid/Defs.lean,Mathlib/Algebra/Group/Submonoid/Membership.lean,Mathlib/Algebra/Group/Submonoid/MulAction.lean,Mathlib/Algebra/Group/Submonoid/Operations.lean,Mathlib/Algebra/Group/Subsemigroup/Basic.lean,Mathlib/Algebra/Group/Subsemigroup/Defs.lean,Mathlib/Algebra/Group/Subsemigroup/Operations.lean,Mathlib/Algebra/Group/Support.lean,Mathlib/Algebra/Group/Units/Defs.lean,Mathlib/Algebra/Module/Equiv/Basic.lean,Mathlib/Algebra/Module/Equiv/Defs.lean,Mathlib/Algebra/Module/LinearMap/Defs.lean,Mathlib/Algebra/Module/LinearMap/Prod.lean,Mathlib/Algebra/Module/Prod.lean,Mathlib/Algebra/Module/Submodule/EqLocus.lean,Mathlib/Algebra/Module/Submodule/Equiv.lean,Mathlib/Algebra/Module/Submodule/Ker.lean,Mathlib/Algebra/Module/Submodule/LinearMap.lean,Mathlib/Algebra/Module/Submodule/Map.lean,Mathlib/Algebra/Module/Submodule/Pointwise.lean,Mathlib/Algebra/Module/Submodule/Range.lean,Mathlib/Algebra/MonoidAlgebra/Grading.lean,Mathlib/Algebra/MonoidAlgebra/MapDomain.lean,Mathlib/Algebra/MonoidAlgebra/ToDirectSum.lean,Mathlib/Algebra/MvPolynomial/Basic.lean,Mathlib/Algebra/MvPolynomial/Comap.lean,Mathlib/Algebra/MvPolynomial/Monad.lean,Mathlib/Algebra/Notation/Prod.lean,Mathlib/Algebra/Order/Quantale.lean,Mathlib/Algebra/Prime/Lemmas.lean,Mathlib/Algebra/Quandle.lean,Mathlib/Algebra/QuaternionBasis.lean,Mathlib/Algebra/Ring/CompTypeclasses.lean,Mathlib/Algebra/Ring/Hom/Defs.lean,Mathlib/Algebra/SkewMonoidAlgebra/Basic.lean,Mathlib/Algebra/Star/Module.lean,Mathlib/Algebra/TrivSqZeroExt.lean,Mathlib/Algebra/Vertex/HVertexOperator.lean,Mathlib/Algebra/Vertex/VertexOperator.lean,Mathlib/Analysis/Analytic/Composition.lean,Mathlib/Analysis/Asymptotics/Defs.lean,Mathlib/Analysis/Asymptotics/Lemmas.lean,Mathlib/Analysis/Asymptotics/Theta.lean,Mathlib/Analysis/CStarAlgebra/CStarMatrix.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Integral.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Order.lean,Mathlib/Analysis/Calculus/ContDiff/Bounds.lean,Mathlib/Analysis/Calculus/Deriv/Mul.lean,Mathlib/Analysis/Calculus/FDeriv/Mul.lean,Mathlib/Analysis/Calculus/FormalMultilinearSeries.lean,Mathlib/Analysis/Convex/Cone/Proper.lean,Mathlib/Analysis/Convex/EGauge.lean,Mathlib/Analysis/Convex/Exposed.lean,Mathlib/Analysis/InnerProductSpace/Adjoint.lean,Mathlib/Analysis/InnerProductSpace/Defs.lean,Mathlib/Analysis/InnerProductSpace/LinearMap.lean,Mathlib/Analysis/InnerProductSpace/Orthonormal.lean,Mathlib/Analysis/InnerProductSpace/PiL2.lean,Mathlib/Analysis/InnerProductSpace/WeakOperatorTopology.lean,Mathlib/Analysis/LocallyConvex/WeakOperatorTopology.lean,Mathlib/Analysis/Normed/Affine/Isometry.lean,Mathlib/Analysis/Normed/Algebra/Basic.lean,Mathlib/Analysis/Normed/Algebra/Spectrum.lean,Mathlib/Analysis/Normed/Lp/lpSpace.lean,Mathlib/Analysis/Normed/Module/Basic.lean,Mathlib/Analysis/Normed/Module/FiniteDimension.lean,Mathlib/Analysis/Normed/Ring/InfiniteSum.lean,Mathlib/Analysis/Normed/Ring/Lemmas.lean,Mathlib/Analysis/NormedSpace/ConformalLinearMap.lean,Mathlib/Analysis/NormedSpace/ENormedSpace.lean,Mathlib/Analysis/NormedSpace/OperatorNorm/Bilinear.lean,Mathlib/Analysis/Seminorm.lean,Mathlib/Analysis/SpecialFunctions/ContinuousFunctionalCalculus/ExpLog.lean,Mathlib/Analysis/SpecificLimits/Basic.lean,Mathlib/CategoryTheory/Action/Concrete.lean,Mathlib/CategoryTheory/GradedObject.lean 343 3 ['github-actions', 'leanprover-community-bot-assistant', 'urkud'] nobody
42-81826
1 month ago
42-81828
1 month ago
2-7052
2 days
23138 grunweg
author:grunweg
feat: (unoriented) bordism groups We define the unoriented bordism group of a topological space and prove that it is an abelian group: we don't prove transitivity of bordisms yet, as that requires the collar neighbourhood theorem and gluing of smooth manifolds, which are both not in mathlib and a sizable piece of work. --- This PR is not ready for review yet; I'm merely opening this to track this branch' state better. In particular, this PR depends on several preliminary PRs: - depends on: #15906 for defining singular n-manifolds - depends on: #23040: define immersions and smooth embeddings: in finite dimensions, these are easy to describe; for mathlib, we will want a correct definition for e.g. Banach manifolds also. - depends on: #22059 defines manifolds with smooth boundary. That PR has two open dependencies; one is slowly getting merged, that other has a few sorries I still need to prove (not difficult). - depends on: #22874 for some constructions - defining unoriented bordisms, and proving some basic constructions about them: will be another PR [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-differential-geometry merge-conflict WIP 1316/3 Mathlib.lean,Mathlib/Geometry/Manifold/Bordisms.lean,Mathlib/Geometry/Manifold/Diffeomorph.lean,Mathlib/Geometry/Manifold/HasSmoothBoundary.lean,Mathlib/Geometry/Manifold/Instances/Real.lean,Mathlib/Geometry/Manifold/IsManifold/Basic.lean,Mathlib/Geometry/Manifold/MFDeriv/SpecificFunctions.lean 7 0 [] nobody
42-30320
1 month ago
80-6601
2 months ago
0-1
1 second
23593 erdOne
author:erdOne
feat(AlgebraicGeometry): the tilde construction is functorial --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebraic-geometry merge-conflict awaiting-author 95/38 Mathlib/AlgebraicGeometry/Modules/Sheaf.lean,Mathlib/AlgebraicGeometry/Modules/Tilde.lean 2 4 ['chrisflav', 'github-actions', 'leanprover-community-bot-assistant'] nobody
42-30006
1 month ago
42-30008
1 month ago
0-71091
19 hours
21065 eric-wieser
author:eric-wieser
feat: generalize `tangentConeAt.lim_zero` to TVS ... and then adjust the `variable`s down the rest of the file to make use of the generality. There are two key lemmas that this does not generalize, which would probably unlock the rest of the file: * `subset_tangentCone_prod_left` (and `_right`) * `zero_mem_tangentCone` --- - [ ] depends on: #20859 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis merge-conflict WIP 55/28 Mathlib/Analysis/Calculus/TangentCone.lean 1 16 ['ADedecker', 'eric-wieser', 'github-actions', 'j-loreaux', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'urkud'] nobody
42-22410
1 month ago
42-22412
1 month ago
23-20319
23 days
22721 grunweg
author:grunweg
chore(MeasureTheory/Function/LpSeminorm/Basic): generalise more results to enorm classes Done for the Carleson project. --- - depends on #22708 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) carleson t-measure-probability merge-conflict WIP 134/10 Mathlib/MeasureTheory/Function/LpSeminorm/Basic.lean 1 2 ['github-actions', 'leanprover-community-bot-assistant'] nobody
41-15078
1 month ago
41-15080
1 month ago
0-6
6 seconds
24354 grunweg
author:grunweg
chore(HasFiniteIntegral): rename three lemmas Discovered in #24343. --- - [ ] depends on: #24343 (to avoid merge conflicts) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-measure-probability merge-conflict 108/30 Mathlib/MeasureTheory/Function/L1Space/HasFiniteIntegral.lean 1 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
41-7039
1 month ago
41-7040
1 month ago
0-4604
1 hour
23791 SEU-Prime
author:SEU-Prime
Create AmiceTrans.lean --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-number-theory merge-conflict WIP 2963/0 Mathlib.lean,Mathlib/Analysis/Normed/Ring/Lemmas2.lean,Mathlib/NumberTheory/Padics/AmiceTrans.lean,Mathlib/NumberTheory/Padics/PSAC.lean,Mathlib/NumberTheory/Padics/PSAC2.lean,Mathlib/NumberTheory/Padics/PSAC3.lean,Mathlib/NumberTheory/Padics/PiGammainPS.lean,Mathlib/NumberTheory/Padics/PsiandVar.lean,Mathlib/RingTheory/AdicCompletion/Lemma.lean,Mathlib/RingTheory/PowerSeries/Comp.lean,Mathlib/Topology/ContinuousMap/ZeroAtBot.lean 11 3 ['SEU-Prime', 'github-actions', 'leanprover-community-bot-assistant'] nobody
40-54359
1 month ago
47-33365
1 month ago
0-0
0 seconds
24091 mattrobball
author:mattrobball
test merge-conflict 97/46 Mathlib/Algebra/Field/Defs.lean,Mathlib/Analysis/Asymptotics/Lemmas.lean,Mathlib/Analysis/LocallyConvex/Basic.lean,Mathlib/Analysis/Normed/Affine/AddTorsor.lean,Mathlib/Analysis/Normed/Module/Basic.lean,Mathlib/Analysis/Normed/Module/Span.lean,Mathlib/Analysis/Normed/MulAction.lean,Mathlib/Analysis/NormedSpace/Pointwise.lean,Mathlib/Dynamics/BirkhoffSum/NormedSpace.lean,Mathlib/MeasureTheory/Function/LpSeminorm/Basic.lean,Mathlib/Topology/ContinuousMap/Compact.lean,Mathlib/Topology/MetricSpace/Holder.lean,Mathlib/Topology/MetricSpace/HolderNorm.lean,docs/overview.yaml,docs/undergrad.yaml 15 5 ['github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'mattrobball'] nobody
40-43777
1 month ago
40-43779
1 month ago
0-0
0 seconds
18771 joelriou
author:joelriou
feat(LinearAlgebra/ExteriorPower): exterior powers of free modules are free Co-authored-by: sophie.morel@ens-lyon.fr --- - [ ] depends on: #18662 - [ ] depends on: #18534 - [ ] depends on: #18651 - [x] depends on: #18590 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict blocked-by-other-PR WIP
label:t-algebra$
1185/160 Mathlib.lean,Mathlib/Analysis/NormedSpace/Multilinear/Curry.lean,Mathlib/Analysis/NormedSpace/PiTensorProduct/ProjectiveSeminorm.lean,Mathlib/Data/Sum/Basic.lean,Mathlib/LinearAlgebra/ExteriorPower/Basic.lean,Mathlib/LinearAlgebra/ExteriorPower/Basis.lean,Mathlib/LinearAlgebra/ExteriorPower/Generators.lean,Mathlib/LinearAlgebra/ExteriorPower/Pairing.lean,Mathlib/LinearAlgebra/Multilinear/Basic.lean,Mathlib/LinearAlgebra/Multilinear/TensorProduct.lean,Mathlib/LinearAlgebra/PiTensorProduct/Basic.lean,Mathlib/LinearAlgebra/PiTensorProduct/Finite.lean,Mathlib/LinearAlgebra/PiTensorProduct/Generators.lean,Mathlib/LinearAlgebra/Span.lean,Mathlib/LinearAlgebra/TensorAlgebra/ToTensorPower.lean,Mathlib/LinearAlgebra/TensorPower/Basic.lean,Mathlib/LinearAlgebra/TensorPower/Pairing.lean,Mathlib/Logic/Function/Basic.lean,Mathlib/RingTheory/PiTensorProduct.lean 19 3 ['alreadydone', 'github-actions', 'mathlib4-dependent-issues-bot'] nobody
40-23621
1 month ago
206-40834
6 months ago
0-0
0 seconds
18735 joelriou
author:joelriou
feat(Algebra/Module): presentation of the exterior power Given a presentation of a `R`-module `M`, we obtain a presentation of `⋀[R]^n M`. --- (Still one sorry left.) - [ ] depends on: #18527 - [ ] depends on: #18432 - [ ] depends on: #18725 - [ ] depends on: #18534 - [ ] depends on: #18662 - [x] depends on: #18590 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict blocked-by-other-PR WIP
label:t-algebra$
1856/157 Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/ExteriorPower.lean,Mathlib/Algebra/Module/Presentation/Basic.lean,Mathlib/Algebra/Module/Presentation/ExteriorPower.lean,Mathlib/Algebra/Module/Presentation/PiTensor.lean,Mathlib/Algebra/Module/Presentation/Tensor.lean,Mathlib/Analysis/NormedSpace/Multilinear/Curry.lean,Mathlib/Analysis/NormedSpace/PiTensorProduct/ProjectiveSeminorm.lean,Mathlib/Data/Sum/Basic.lean,Mathlib/LinearAlgebra/ExteriorPower/Basic.lean,Mathlib/LinearAlgebra/ExteriorPower/Generators.lean,Mathlib/LinearAlgebra/Multilinear/Basic.lean,Mathlib/LinearAlgebra/Multilinear/TensorProduct.lean,Mathlib/LinearAlgebra/PiTensorProduct/Basic.lean,Mathlib/LinearAlgebra/PiTensorProduct/Finite.lean,Mathlib/LinearAlgebra/PiTensorProduct/Generators.lean,Mathlib/LinearAlgebra/Span.lean,Mathlib/LinearAlgebra/TensorPower.lean,Mathlib/Logic/Function/Basic.lean,Mathlib/RingTheory/PiTensorProduct.lean 20 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
40-23618
1 month ago
206-40836
6 months ago
0-0
0 seconds
18662 joelriou
author:joelriou
feat(LinearAlgebra/ExteriorPower): generators of the exterior powers --- - [ ] depends on: #18534 - [x] depends on: #18590 - [ ] depends on: #18725 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict blocked-by-other-PR WIP
label:t-algebra$
818/158 Mathlib.lean,Mathlib/Analysis/NormedSpace/Multilinear/Curry.lean,Mathlib/Analysis/NormedSpace/PiTensorProduct/ProjectiveSeminorm.lean,Mathlib/Data/Sum/Basic.lean,Mathlib/LinearAlgebra/ExteriorPower/Basic.lean,Mathlib/LinearAlgebra/ExteriorPower/Generators.lean,Mathlib/LinearAlgebra/Multilinear/Basic.lean,Mathlib/LinearAlgebra/Multilinear/TensorProduct.lean,Mathlib/LinearAlgebra/PiTensorProduct/Basic.lean,Mathlib/LinearAlgebra/PiTensorProduct/Finite.lean,Mathlib/LinearAlgebra/PiTensorProduct/Generators.lean,Mathlib/LinearAlgebra/Span.lean,Mathlib/LinearAlgebra/TensorPower.lean,Mathlib/Logic/Function/Basic.lean,Mathlib/RingTheory/PiTensorProduct.lean 15 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
40-23614
1 month ago
206-40838
6 months ago
0-0
0 seconds
18551 joelriou
author:joelriou
feat(AlgebraicGeometry): the algebraic De Rham complex If `B` is an `A`-algebra, we construct the algebraic De Rham complex of `B` over `A`: it is a cochain complex of `A`-modules. --- - [ ] depends on: #18735 - [ ] depends on: #18662 - [ ] depends on: #18725 - [ ] depends on: #18534 - [ ] depends on: #18527 - [x] depends on: #18440 - [ ] depends on: #18432 - [x] depends on: #18408 - [x] depends on: #18389 - [x] depends on: #18374 - [x] depends on: #18359 - [x] depends on: #18332 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-algebraic-geometry merge-conflict blocked-by-other-PR WIP
label:t-algebra$
2836/156 Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/ExteriorPower.lean,Mathlib/Algebra/Module/Presentation/Basic.lean,Mathlib/Algebra/Module/Presentation/Cokernel.lean,Mathlib/Algebra/Module/Presentation/Differentials.lean,Mathlib/Algebra/Module/Presentation/DirectSum.lean,Mathlib/Algebra/Module/Presentation/ExteriorPower.lean,Mathlib/Algebra/Module/Presentation/PiTensor.lean,Mathlib/Algebra/Module/Presentation/RestrictScalars.lean,Mathlib/Algebra/Module/Presentation/Tensor.lean,Mathlib/Analysis/NormedSpace/Multilinear/Curry.lean,Mathlib/Analysis/NormedSpace/PiTensorProduct/ProjectiveSeminorm.lean,Mathlib/Data/Finsupp/Defs.lean,Mathlib/Data/Sum/Basic.lean,Mathlib/LinearAlgebra/ExteriorPower/Basic.lean,Mathlib/LinearAlgebra/ExteriorPower/Generators.lean,Mathlib/LinearAlgebra/Multilinear/Basic.lean,Mathlib/LinearAlgebra/Multilinear/TensorProduct.lean,Mathlib/LinearAlgebra/PiTensorProduct/Basic.lean,Mathlib/LinearAlgebra/PiTensorProduct/Finite.lean,Mathlib/LinearAlgebra/PiTensorProduct/Generators.lean,Mathlib/LinearAlgebra/Span.lean,Mathlib/LinearAlgebra/TensorPower.lean,Mathlib/Logic/Function/Basic.lean,Mathlib/RingTheory/DeRham/Basic.lean,Mathlib/RingTheory/PiTensorProduct.lean 26 n/a ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
40-23612
1 month ago
unknown
unknown
14731 adomani
author:adomani
feat: the repeated typeclass assumption linter [#mathlib4 > recyclable variables @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/recyclable.20variables/near/451167963) also [#mathlib4 > Normed modules @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Normed.20modules/near/512242167) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-linter merge-conflict WIP 178/0 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter.lean,Mathlib/Tactic/Linter/DependentTypeclass.lean,MathlibTest/DependentTypeclass.lean 5 3 ['github-actions', 'leanprover-community-bot-assistant', 'mattrobball'] nobody
40-20317
1 month ago
52-37719
1 month ago
0-109
1 minute
24140 mattrobball
author:mattrobball
test merge-conflict 176/91 Mathlib/Algebra/Group/Defs.lean,Mathlib/Algebra/GroupWithZero/Defs.lean,Mathlib/Algebra/Ring/Defs.lean,Mathlib/AlgebraicGeometry/AffineSpace.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Affine.lean,Mathlib/Analysis/CStarAlgebra/Classes.lean,Mathlib/Data/Complex/Module.lean,Mathlib/LinearAlgebra/Matrix/Charpoly/Coeff.lean,Mathlib/NumberTheory/NumberField/ProductFormula.lean,Mathlib/RingTheory/Algebraic/Integral.lean,Mathlib/RingTheory/LaurentSeries.lean,Mathlib/RingTheory/Localization/Integral.lean,Mathlib/RingTheory/RingHom/Unramified.lean,Mathlib/RingTheory/Spectrum/Prime/ChevalleyComplexity.lean,Mathlib/RingTheory/Valuation/Basic.lean,Mathlib/RingTheory/Valuation/ValuationSubring.lean,Mathlib/Topology/Algebra/Valued/WithVal.lean 17 5 ['github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'mattrobball'] nobody
40-18780
1 month ago
40-18782
1 month ago
0-0
0 seconds
18527 joelriou
author:joelriou
feat(Algebra/Module): presentation of the `PiTensorProduct` Given a presentation of a finite number of `R`-modules `M i`, we obtain a presentation of the module `⨂[R] i, M i`. --- - [x] depends on: #18408 - [ ] depends on: #18432 - [ ] depends on: #18725 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict blocked-by-other-PR WIP
label:t-algebra$
504/4 Mathlib.lean,Mathlib/Algebra/Module/Presentation/PiTensor.lean,Mathlib/Analysis/NormedSpace/PiTensorProduct/ProjectiveSeminorm.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 8 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
38-15866
1 month ago
38-15868
1 month ago
0-0
0 seconds
13649 FR-vdash-bot
author:FR-vdash-bot
chore: redefine `Nat.div2` `Nat.bodd` The new definitions are faster than the old ones. `Nat.binaryRec` will be moved to batteries (https://github.com/leanprover-community/batteries/pull/799) or core (https://github.com/leanprover/lean4/pull/3756), so relevant contents are moved to a new file temporarily. --- - [x] depends on: #15567 - [x] depends on: #19666 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict 63/88 Mathlib/Computability/Primrec.lean,Mathlib/Data/Int/Bitwise.lean,Mathlib/Data/Nat/Bits.lean,Mathlib/Data/Nat/Bitwise.lean,Mathlib/Data/Nat/Size.lean,Mathlib/Logic/Denumerable.lean,Mathlib/Logic/Encodable/Basic.lean,Mathlib/Logic/Equiv/Nat.lean 8 15 ['FR-vdash-bot', 'digama0', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'urkud'] digama0
assignee:digama0
37-72585
1 month ago
37-72587
1 month ago
87-51692
87 days
22856 mattrobball
author:mattrobball
test merge-conflict 8/2 Mathlib/Algebra/Algebra/Defs.lean,Mathlib/Analysis/Complex/Hadamard.lean,Mathlib/Analysis/RCLike/Inner.lean,Mathlib/FieldTheory/Galois/Profinite.lean 4 5 ['github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'mattrobball'] nobody
37-60146
1 month ago
37-60148
1 month ago
0-0
0 seconds
23635 FLDutchmann
author:FLDutchmann
feat(NumberTheory/SelbergSieve): define Selberg's weights and prove basic results. This PR defines weights used by Selberg's lambda squared sieve. Though we don't prove it, these weights minimise the main sum under the constraint that the weights are supported up to $\sqrt{y}$. --- - [ ] depends on: #22052 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis t-number-theory merge-conflict blocked-by-other-PR 403/1 Mathlib/Data/Nat/GCD/Basic.lean,Mathlib/NumberTheory/Divisors.lean,Mathlib/NumberTheory/SelbergSieve.lean 3 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
37-60022
1 month ago
37-60023
1 month ago
0-18
18 seconds
23872 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.) --- - [ ] depends on: #23364 - [ ] depends on: #22205 - [ ] depends on: #21032 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory merge-conflict blocked-by-other-PR WIP 1222/367 Mathlib.lean,Mathlib/Algebra/Category/Grp/Basic.lean,Mathlib/Algebra/Category/Grp/FilteredColimits.lean,Mathlib/Algebra/Category/ModuleCat/FilteredColimits.lean,Mathlib/Algebra/Category/MonCat/Basic.lean,Mathlib/Algebra/Category/MonCat/FilteredColimits.lean,Mathlib/Algebra/Category/Ring/Basic.lean,Mathlib/Algebra/Category/Ring/FilteredColimits.lean,Mathlib/CategoryTheory/Limits/Final.lean,Mathlib/CategoryTheory/Limits/FintypeCat.lean,Mathlib/CategoryTheory/Limits/IsConnected.lean,Mathlib/CategoryTheory/Limits/Preserves/Shapes/Multiequalizer.lean,Mathlib/CategoryTheory/Limits/Preserves/Ulift.lean,Mathlib/CategoryTheory/Limits/Shapes/Multiequalizer.lean,Mathlib/CategoryTheory/Limits/Shapes/MultiequalizerPullback.lean,Mathlib/CategoryTheory/Limits/Shapes/SingleObj.lean,Mathlib/CategoryTheory/Limits/Types/ColimitType.lean,Mathlib/CategoryTheory/Limits/Types/Colimits.lean,Mathlib/CategoryTheory/Limits/Types/Filtered.lean,Mathlib/CategoryTheory/Limits/Types/Multicoequalizer.lean,Mathlib/CategoryTheory/Types.lean,Mathlib/Order/CompleteLattice/MulticoequalizerDiagram.lean,Mathlib/Topology/Category/TopCat/Limits/Basic.lean 23 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
37-59898
1 month ago
37-59899
1 month ago
0-0
0 seconds
24275 joelriou
author:joelriou
feat(Algebra/Homology): the canonical t-structure on the derived category --- - [x] depends on: #22574 - [ ] depends on: #24191 - [ ] depends on: #24276 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory merge-conflict blocked-by-other-PR WIP 909/191 Mathlib.lean,Mathlib/Algebra/Homology/DerivedCategory/Basic.lean,Mathlib/Algebra/Homology/DerivedCategory/TStructure.lean,Mathlib/Algebra/Homology/Embedding/CochainComplex.lean,Mathlib/Algebra/Homology/Embedding/ComplementaryTrunc.lean,Mathlib/Algebra/Homology/Embedding/TruncLEHomology.lean,Mathlib/CategoryTheory/ObjectProperty/ContainsZero.lean,Mathlib/CategoryTheory/ObjectProperty/Shift.lean,Mathlib/CategoryTheory/Triangulated/HomologicalFunctor.lean,Mathlib/CategoryTheory/Triangulated/Subcategory.lean,Mathlib/CategoryTheory/Triangulated/TStructure/Basic.lean 11 4 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
37-59772
1 month ago
37-59773
1 month ago
0-0
0 seconds
24549 grunweg
author:grunweg
feat: define embedded submanifolds, attempt 1 Not meant to be merged (I think a different design is better); opening this so I can find this more easily. --- - [ ] depends on: #23040 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-differential-geometry merge-conflict blocked-by-other-PR WIP 1445/2 Mathlib.lean,Mathlib/Analysis/NormedSpace/HahnBanach/Splits.lean,Mathlib/Geometry/Manifold/Diffeomorph.lean,Mathlib/Geometry/Manifold/EmbeddedSubmanifold.lean,Mathlib/Geometry/Manifold/IsImmersionEmbedding.lean,Mathlib/Geometry/Manifold/LocalDiffeomorph.lean,Mathlib/Geometry/Manifold/MSplits.lean,Mathlib/LinearAlgebra/Prod.lean 8 2 ['leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
37-45530
1 month ago
37-45530
1 month ago
0-1
1 second
23921 alreadydone
author:alreadydone
Jyxu/projective trace --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict WIP
label:t-algebra$
157/123 Mathlib/FieldTheory/CardinalEmb.lean,Mathlib/FieldTheory/Relrank.lean,Mathlib/LinearAlgebra/Contraction.lean,Mathlib/LinearAlgebra/Dual.lean,Mathlib/RingTheory/LocalProperties/Projective.lean 5 1 ['leanprover-community-bot-assistant'] nobody
37-45362
1 month ago
37-45362
1 month ago
0-0
0 seconds
21252 ADedecker
author:ADedecker
feat: redefine uniformly convex normed spaces with filters instead of epsilons And conceptualize some proofs. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-topology merge-conflict
label:t-algebra$
301/87 Mathlib/Analysis/Convex/Uniform.lean,Mathlib/Analysis/InnerProductSpace/Basic.lean,Mathlib/Order/Basic.lean,Mathlib/Order/Filter/Pointwise.lean,Mathlib/Topology/Algebra/UniformGroup/Defs.lean,Mathlib/Topology/Algebra/UniformMulAction.lean 6 1 ['github-actions'] nobody
37-45101
1 month ago
37-45101
1 month ago
0-0
0 seconds
20201 dagurtomas
author:dagurtomas
feat(AlgebraicTopology): anodyne morphisms of simplicial sets --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology merge-conflict WIP 148/0 Mathlib.lean,Mathlib/AlgebraicTopology/Anodyne.lean,Mathlib/AlgebraicTopology/KanFibration.lean,Mathlib/CategoryTheory/MorphismProperty/WeakSaturation.lean 4 1 ['github-actions'] nobody
37-44931
1 month ago
37-44931
1 month ago
0-0
0 seconds
19821 eric-wieser
author:eric-wieser
feat: add a Qq version of AtomM that groups by type --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-meta merge-conflict WIP 332/30 Mathlib/Data/Ineq.lean,Mathlib/Tactic/Linarith/Datatypes.lean,Mathlib/Tactic/Linarith/Oracle/SimplexAlgorithm.lean,Mathlib/Tactic/Linarith/Preprocessing.lean,Mathlib/Util/AtomM.lean,Mathlib/Util/Qq.lean 6 1 ['github-actions'] nobody
37-44914
1 month ago
37-44914
1 month ago
0-0
0 seconds
19520 erdOne
author:erdOne
refactor(Algebra/Module): Redefine `LocalizedModule` in terms of `OreLocalization` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict
label:t-algebra$
610/493 Mathlib.lean,Mathlib/Algebra/Module/LocalizedModule/Basic.lean,Mathlib/AlgebraicGeometry/AffineScheme.lean,Mathlib/AlgebraicGeometry/Modules/Tilde.lean,Mathlib/AlgebraicGeometry/OpenImmersion.lean,Mathlib/GroupTheory/OreLocalization/Basic.lean,Mathlib/RingTheory/Localization/BaseChange.lean,Mathlib/RingTheory/OreLocalization/Basic.lean,Mathlib/RingTheory/OreLocalization/Module.lean,Mathlib/RingTheory/OreLocalization/Ring.lean 10 1 ['github-actions'] nobody
37-44903
1 month ago
37-44903
1 month ago
8-56155
8 days
19120 hrmacbeth
author:hrmacbeth
feat: stop `ring`/`abel` from seeing algebraic operations inside `let`s This draft PR illustrates a feature I would like to see in core: a variant of `whnf` which allows particular kinds of reduction, such as zeta-delta reduction, to be turned off. Here it is used to make ring-normalization and abelian-group-normalization a bit more responsive to what (I think) users expect: these normalizations would no longer look inside user-defined lets to see algebraic operations in those expressions. Note: In Lean/Mathlib 3, `ring` matched for algebraic operations on an algebraic expression `e` itself, not on `← whnfR e`. So mathlib3 `ring` didn't see algebraic operations inside `let`s -- but it also didn't see algebraic operations requiring beta-reduction (like `(fun t ↦ t + 1) x`) or see inside abbreviations. [Zulip](https://leanprover.zulipchat.com/#narrow/channel/239415-metaprogramming-.2F-tactics/topic/whnf.20variant.20which.20preserves.20let-bindings) Update: fortuitously, it looks like the new core PR https://github.com/leanprover/lean4/pull/6053 will provide this feature! --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta merge-conflict blocked-by-core-PR 137/15 Archive/Imo/Imo2006Q3.lean,Archive/Imo/Imo2008Q2.lean,Mathlib.lean,Mathlib/Algebra/ContinuedFractions/Computation/Approximations.lean,Mathlib/Analysis/Analytic/Composition.lean,Mathlib/Analysis/Calculus/FDeriv/Measurable.lean,Mathlib/Analysis/SpecialFunctions/Gamma/BohrMollerup.lean,Mathlib/Analysis/SpecialFunctions/Integrals.lean,Mathlib/Analysis/SpecialFunctions/Stirling.lean,Mathlib/Data/Real/Pi/Irrational.lean,Mathlib/NumberTheory/LSeries/HurwitzZetaOdd.lean,Mathlib/NumberTheory/SumPrimeReciprocals.lean,Mathlib/RingTheory/WittVector/DiscreteValuationRing.lean,Mathlib/Tactic/Abel.lean,Mathlib/Tactic/Polyrith.lean,Mathlib/Tactic/Ring/Basic.lean,Mathlib/Tactic/Ring/RingNF.lean,Mathlib/Topology/MetricSpace/GromovHausdorff.lean,Mathlib/Util/WHNF.lean,MathlibTest/abel.lean,MathlibTest/ring.lean 21 5 ['JovanGerb', 'github-actions', 'grunweg', 'hrmacbeth'] nobody
37-44894
1 month ago
37-44894
1 month ago
0-0
0 seconds
17069 yuma-mizuno
author:yuma-mizuno
chore(CategoryTheory/Functor/Basic): put `simp` at `Functor.id_comp` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory merge-conflict 41/30 Mathlib/CategoryTheory/Adjunction/Mates.lean,Mathlib/CategoryTheory/Functor/Basic.lean,Mathlib/CategoryTheory/GuitartExact/VerticalComposition.lean,Mathlib/CategoryTheory/Limits/HasLimits.lean,Mathlib/CategoryTheory/Shift/CommShift.lean 5 3 ['github-actions', 'leanprover-bot', 'yuma-mizuno'] nobody
37-44884
1 month ago
37-44884
1 month ago
0-0
0 seconds
15024 mattrobball
author:mattrobball
chore(Algebra.Basic): scope and rename universal `Nat`-algebra and `Int`-algebra instances We rename `algebraNat` to `Nat.instAlgebraOfSemiring` and `algebraInt` to `Int.instAlgebraOfRing` to be consistent with existing naming conventions. We also scope them to avoid typeclass search tripping over them unnecessarily. --- Moves: - algebraNat -> Nat.instAlgebraOfSemiring - algebraInt -> Int.instAlgebraOfRing [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict
label:t-algebra$
178/27 Archive/Wiedijk100Theorems/AbelRuffini.lean,Counterexamples/Pseudoelement.lean,Mathlib/Algebra/Algebra/Basic.lean,Mathlib/Algebra/Algebra/Hom.lean,Mathlib/Algebra/Algebra/Subalgebra/Basic.lean,Mathlib/Algebra/Algebra/Subalgebra/Unitization.lean,Mathlib/Algebra/Category/ModuleCat/Injective.lean,Mathlib/Algebra/FreeAlgebra.lean,Mathlib/Algebra/Module/Bimodule.lean,Mathlib/Algebra/Module/Zlattice/Basic.lean,Mathlib/Algebra/MvPolynomial/Counit.lean,Mathlib/Algebra/MvPolynomial/Supported.lean,Mathlib/Algebra/Polynomial/AlgebraMap.lean,Mathlib/Algebra/Polynomial/DenomsClearable.lean,Mathlib/Algebra/Polynomial/UnitTrinomial.lean,Mathlib/Algebra/RingQuot.lean,Mathlib/Analysis/Complex/UpperHalfPlane/Basic.lean,Mathlib/Analysis/Complex/UpperHalfPlane/Metric.lean,Mathlib/Analysis/Complex/UpperHalfPlane/Topology.lean,Mathlib/Data/Matrix/Kronecker.lean,Mathlib/Data/Real/Irrational.lean,Mathlib/FieldTheory/IsAlgClosed/Classification.lean,Mathlib/LinearAlgebra/CliffordAlgebra/Basic.lean,Mathlib/LinearAlgebra/FreeModule/IdealQuotient.lean,Mathlib/LinearAlgebra/FreeProduct/Basic.lean,Mathlib/LinearAlgebra/Matrix/Adjugate.lean,Mathlib/LinearAlgebra/QuadraticForm/Basic.lean,Mathlib/LinearAlgebra/TensorAlgebra/Basic.lean,Mathlib/NumberTheory/ClassNumber/AdmissibleCardPowDegree.lean,Mathlib/NumberTheory/ClassNumber/Finite.lean,Mathlib/NumberTheory/Cyclotomic/Basic.lean,Mathlib/NumberTheory/Cyclotomic/Discriminant.lean,Mathlib/NumberTheory/Cyclotomic/Rat.lean,Mathlib/NumberTheory/FLT/Three.lean,Mathlib/NumberTheory/LegendreSymbol/QuadraticChar/GaussSum.lean,Mathlib/NumberTheory/Liouville/Basic.lean,Mathlib/NumberTheory/Liouville/LiouvilleNumber.lean,Mathlib/NumberTheory/Modular.lean,Mathlib/NumberTheory/ModularForms/EisensteinSeries/Defs.lean,Mathlib/NumberTheory/ModularForms/Identities.lean,Mathlib/NumberTheory/ModularForms/JacobiTheta/OneVariable.lean,Mathlib/NumberTheory/ModularForms/SlashActions.lean,Mathlib/NumberTheory/ModularForms/SlashInvariantForms.lean,Mathlib/NumberTheory/MulChar/Lemmas.lean,Mathlib/NumberTheory/NumberField/Basic.lean,Mathlib/NumberTheory/NumberField/CanonicalEmbedding/Basic.lean,Mathlib/NumberTheory/NumberField/ClassNumber.lean,Mathlib/NumberTheory/NumberField/Discriminant.lean,Mathlib/NumberTheory/NumberField/Embeddings.lean,Mathlib/NumberTheory/NumberField/FractionalIdeal.lean,Mathlib/NumberTheory/NumberField/Norm.lean,Mathlib/NumberTheory/NumberField/Units/DirichletTheorem.lean,Mathlib/RepresentationTheory/Maschke.lean,Mathlib/RingTheory/Adjoin/Basic.lean,Mathlib/RingTheory/Adjoin/FG.lean,Mathlib/RingTheory/AlgebraTower.lean,Mathlib/RingTheory/Discriminant.lean,Mathlib/RingTheory/FractionalIdeal/Norm.lean,Mathlib/RingTheory/Ideal/Norm.lean,Mathlib/RingTheory/IntegralClosure/IsIntegralClosure/Basic.lean,Mathlib/RingTheory/Localization/Basic.lean,Mathlib/RingTheory/Localization/FractionRing.lean,Mathlib/RingTheory/Polynomial/Cyclotomic/Eval.lean,Mathlib/RingTheory/Polynomial/Cyclotomic/Expand.lean,Mathlib/RingTheory/Polynomial/Cyclotomic/Roots.lean,Mathlib/RingTheory/Polynomial/GaussLemma.lean,Mathlib/RingTheory/Polynomial/Hermite/Gaussian.lean,Mathlib/RingTheory/Polynomial/Pochhammer.lean,Mathlib/RingTheory/RootsOfUnity/Lemmas.lean,Mathlib/RingTheory/RootsOfUnity/Minpoly.lean,Mathlib/RingTheory/TensorProduct/Basic.lean,Mathlib/RingTheory/Trace/Basic.lean,Mathlib/RingTheory/WittVector/Basic.lean,Mathlib/RingTheory/WittVector/Defs.lean,Mathlib/RingTheory/WittVector/Frobenius.lean,Mathlib/RingTheory/WittVector/InitTail.lean,Mathlib/RingTheory/WittVector/IsPoly.lean,Mathlib/RingTheory/WittVector/MulP.lean,Mathlib/RingTheory/WittVector/StructurePolynomial.lean,Mathlib/RingTheory/WittVector/Verschiebung.lean 80 6 ['eric-wieser', 'github-actions', 'leanprover-bot', 'mattrobball'] nobody
37-44873
1 month ago
37-44873
1 month ago
0-0
0 seconds
14803 StevenClontz
author:StevenClontz
chore: use `Disjoint` nhd filters for all separation axioms --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology merge-conflict 157/122 Mathlib/Topology/Separation.lean 1 1 ['github-actions'] nobody
37-44868
1 month ago
37-44869
1 month ago
0-0
0 seconds
14675 adomani
author:adomani
dev: the repeated variable linter --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-linter merge-conflict WIP 71/0 Mathlib/Tactic/Linter/Lint.lean 1 1 ['github-actions'] nobody
37-44863
1 month ago
37-44863
1 month ago
0-8
8 seconds
14330 Ruben-VandeVelde
author:Ruben-VandeVelde
chore: split Mathlib.Algebra.Star.Basic --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict awaiting-author 446/331 Mathlib.lean,Mathlib/Algebra/Module/LinearMap/Star.lean,Mathlib/Algebra/Star/Basic.lean,Mathlib/Algebra/Star/BigOperators.lean,Mathlib/Algebra/Star/Defs.lean,Mathlib/Algebra/Star/Lemmas.lean,Mathlib/Algebra/Star/Order.lean,Mathlib/Algebra/Star/Pi.lean,Mathlib/Algebra/Star/Pointwise.lean,Mathlib/Algebra/Star/Rat.lean,Mathlib/Algebra/Star/Regular.lean,Mathlib/Algebra/Star/StarRingHom.lean,Mathlib/Analysis/NormedSpace/LinearIsometry.lean,Mathlib/Data/Complex/Basic.lean,scripts/noshake.json 15 3 ['github-actions', 'grunweg', 'j-loreaux'] nobody
37-44823
1 month ago
37-44849
1 month ago
0-45204
12 hours
14137 mattrobball
author:mattrobball
chore(Algebra.Basic): postpone importing algebra instances for `Nat`, `Int`, and `Rat` This should help typeclass synthesis by avoiding these instances unless absolutely necessary. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict 678/356 Counterexamples/Pseudoelement.lean,Mathlib.lean,Mathlib/Algebra/Algebra/Basic.lean,Mathlib/Algebra/Algebra/Bilinear.lean,Mathlib/Algebra/Algebra/Equiv.lean,Mathlib/Algebra/Algebra/Hom/Basic.lean,Mathlib/Algebra/Algebra/Hom/Int.lean,Mathlib/Algebra/Algebra/Hom/Nat.lean,Mathlib/Algebra/Algebra/Hom/Rat.lean,Mathlib/Algebra/Algebra/Int.lean,Mathlib/Algebra/Algebra/Nat.lean,Mathlib/Algebra/Algebra/NonUnitalHom.lean,Mathlib/Algebra/Algebra/NonUnitalSubalgebra.lean,Mathlib/Algebra/Algebra/Prod.lean,Mathlib/Algebra/Algebra/Rat.lean,Mathlib/Algebra/Algebra/Subalgebra/Basic.lean,Mathlib/Algebra/Algebra/Subalgebra/Int.lean,Mathlib/Algebra/Algebra/Subalgebra/Nat.lean,Mathlib/Algebra/Algebra/Subalgebra/Unitization.lean,Mathlib/Algebra/Algebra/Tower.lean,Mathlib/Algebra/FreeAlgebra.lean,Mathlib/Algebra/Group/AddChar.lean,Mathlib/Algebra/Module/Bimodule.lean,Mathlib/Algebra/Module/Zlattice/Basic.lean,Mathlib/Algebra/MonoidAlgebra/Basic.lean,Mathlib/Algebra/MvPolynomial/Counit.lean,Mathlib/Algebra/MvPolynomial/NatInt.lean,Mathlib/Algebra/MvPolynomial/Supported.lean,Mathlib/Algebra/Polynomial/AlgebraMap.lean,Mathlib/Algebra/Polynomial/DenomsClearable.lean,Mathlib/Algebra/Polynomial/Int.lean,Mathlib/Algebra/RingQuot.lean,Mathlib/Analysis/NormedSpace/Basic.lean,Mathlib/CategoryTheory/Galois/Examples.lean,Mathlib/Data/Complex/Module.lean,Mathlib/Data/Real/Irrational.lean,Mathlib/FieldTheory/IsAlgClosed/AlgebraicClosure.lean,Mathlib/FieldTheory/SplittingField/Construction.lean,Mathlib/LinearAlgebra/Matrix/Adjugate.lean,Mathlib/LinearAlgebra/Prod.lean,Mathlib/NumberTheory/ClassNumber/AdmissibleAbs.lean,Mathlib/NumberTheory/NumberField/Basic.lean,Mathlib/NumberTheory/NumberField/Embeddings.lean,Mathlib/RingTheory/Adjoin/Basic.lean,Mathlib/RingTheory/Adjoin/FG.lean,Mathlib/RingTheory/Adjoin/NatInt.lean,Mathlib/RingTheory/AlgebraTower.lean,Mathlib/RingTheory/Bialgebra/Hom.lean,Mathlib/RingTheory/Coalgebra/Hom.lean,Mathlib/RingTheory/IntegralClosure.lean,Mathlib/RingTheory/Localization/Basic.lean,Mathlib/RingTheory/Localization/FractionRing.lean,Mathlib/RingTheory/Localization/FractionRingInt.lean,Mathlib/RingTheory/Localization/Int.lean,Mathlib/RingTheory/Localization/Nat.lean,Mathlib/RingTheory/Polynomial/GaussLemma.lean,Mathlib/RingTheory/Polynomial/Pochhammer.lean,Mathlib/RingTheory/PowerSeries/WellKnown.lean,Mathlib/RingTheory/TensorProduct/Basic.lean,Mathlib/RingTheory/WittVector/MulCoeff.lean,Mathlib/Topology/Algebra/Algebra.lean,Mathlib/Topology/Instances/Real.lean,test/infer_instance.lean,test/instance_diamonds.lean 64 7 ['fpvandoorn', 'github-actions', 'grunweg', 'leanprover-bot', 'mattrobball'] nobody
37-44778
1 month ago
327-40374
10 months ago
0-0
0 seconds
14023 mattrobball
author:mattrobball
perf(RingTheory.OreLocalization): make data irreducible We generally do not want to unfold operations passing through `Quotient` if we can avoid it for performance reasons. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict 43/32 Mathlib/GroupTheory/MonoidLocalization.lean,Mathlib/RingTheory/OreLocalization/Basic.lean,Mathlib/RingTheory/OreLocalization/Ring.lean 3 5 ['github-actions', 'grunweg', 'leanprover-bot', 'mattrobball'] nobody
37-44718
1 month ago
345-34541
11 months ago
0-0
0 seconds
14007 adomani
author:adomani
test: papercut linter working on all mathlib This PR is a testing ground for potential issues with the papercut linter #13999. It is not intended to be merged. The linter is active on all of mathlib, to make sure that the linter does not throw errors, but only emits warnings! --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-linter merge-conflict WIP 249/0 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter.lean,Mathlib/Tactic/Linter/Papercut.lean,test/Papercut.lean 5 1 ['github-actions'] nobody
37-44708
1 month ago
37-44708
1 month ago
0-0
0 seconds
20354 eric-wieser
author:eric-wieser
feat: generalize `ContinuousLinearMap.curry` to TVS Follow on from #10777 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis merge-conflict 57/25 Mathlib/Analysis/NormedSpace/Multilinear/Curry.lean 1 3 ['eric-wieser', 'github-actions', 'leanprover-community-bot-assistant'] nobody
37-44643
1 month ago
37-44643
1 month ago
0-0
0 seconds
11523 thorimur
author:thorimur
bench: test syntax linter --- The purpose of this PR is just to bench the "best-case scenario" for a linter which iterates through syntax, updating and checking a simple counter along the way. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-linter merge-conflict 22/0 Mathlib.lean,Mathlib/Command/Linter.lean,Mathlib/Tactic/Common.lean 3 3 ['grunweg', 'leanprover-bot', 'thorimur'] nobody
37-44552
1 month ago
37-44552
1 month ago
0-0
0 seconds
8511 eric-wieser
author:eric-wieser
refactor(MeasureTheory/Measure/Haar/Basic): partially generalize to the affine case Without a `Mul` version of `AddTorsor`, this generalization can only go so far. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-measure-probability merge-conflict awaiting-author 52/46 Mathlib/MeasureTheory/Measure/Haar/Basic.lean 1 0 [] nobody
37-44454
1 month ago
37-44454
1 month ago
0-0
0 seconds
7994 ericrbg
author:ericrbg
chore: generalize `LieSubalgebra.mem_map_submodule` --- Not sure if we should rename to something like `mem_map_iff_mem_map_submodule` or not. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict please-adopt
label:t-algebra$
16/4 Mathlib/Algebra/Lie/SkewAdjoint.lean,Mathlib/Algebra/Lie/Subalgebra.lean 2 3 ['eric-wieser', 'ericrbg'] nobody
37-44442
1 month ago
37-44442
1 month ago
0-0
0 seconds
6317 eric-wieser
author:eric-wieser
refactor(Data/Finsupp/Defs): make Finsupp.single defeq to Pi.single By adding a `DecidableEq ι` argument to `Finsupp.single`, we remove the reference to `Classical.decEq ι` in the definition, which in turn means that when coerced to a function it is now defeq to `Pi.single`. This also brings it in line with `DFinsupp.single`. This does not go as far as making `Finsupp.single` computable. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data merge-conflict WIP 269/226 Mathlib/Algebra/BigOperators/Finsupp.lean,Mathlib/Data/Finsupp/AList.lean,Mathlib/Data/Finsupp/Basic.lean,Mathlib/Data/Finsupp/Defs.lean,Mathlib/Data/Finsupp/Fintype.lean,Mathlib/Data/Finsupp/Indicator.lean,Mathlib/Data/Finsupp/Multiset.lean,Mathlib/Data/Finsupp/Order.lean,Mathlib/Data/Finsupp/ToDFinsupp.lean,Mathlib/Data/Nat/Choose/Multinomial.lean,Mathlib/LinearAlgebra/Basis.lean,Mathlib/LinearAlgebra/Finsupp.lean 12 0 [] nobody
37-44436
1 month ago
37-44436
1 month ago
0-0
0 seconds
6277 jjaassoonn
author:jjaassoonn
Dimension theory Some results are - The ring Krull dimension and the topological dimension of the prime spectrum of a ring are the same - A field is zero-dimensional and a PID that is not a field is one dimensional - An Artinian ring is zero-dimensional - The Krull dimension of ring $R$ is equal to the supremum of heights of maximal ideals [00KG](https://stacks.math.columbia.edu/tag/00KG) - two definitions of module length agree - A module is finite length iff both artinian and noetherian - length of module $M$ is equal to the sum of length of $N$ and length of $M / N$ where $N$ is a submodule of $M$. - Noetherian ring has only finitely many minimal primes #9088 - In a zero dimensional ring, prime ideals are maximal - Artinian rings has finitely many maximal ideals #9087 - zero-dimensional rings with finitely many prime ideals are products of its localizations: $R \cong \prod_{\mathfrak{p}}R_{\mathfrak{p}}$ - Let $M_0 \le ... \le M_n$, then $l(M_n/ M_0) = l(M_1/M_0) + l(M_2/M_1) + ... + l(M_n/M_{n-1})$ where $l$ denotes module length. - If $f : R \to S$ is a ring homomorphism and $M$ an $S$-module, then $l_R(M) \le l_S(M)$, when $f$ is surjective then they are equal. (Note that this is expressed using `[Algebra R S]` and `RestrictScalars R S M`, instead of a literal ring hom) - Artinian rings are noetherian ring of dimension 0. - For 0-dimensional local ring, its maximal ideal is locally nilpotent - In notherian ring, $I \le \sqrt{J}$ implies $I ^ n \le J$ for some $n$ --- - [x] depends on: #6309 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict
label:t-algebra$
3289/459 Mathlib.lean,Mathlib/Algebra/Module/Length.lean,Mathlib/Algebra/Module/Submodule/JordanHolder.lean,Mathlib/Algebra/PUnitInstances.lean,Mathlib/AlgebraicGeometry/PrimeSpectrum/ArtinianAndNoetherian.lean,Mathlib/Data/List/Basic.lean,Mathlib/Data/List/Dedup.lean,Mathlib/Data/List/Nodup.lean,Mathlib/LinearAlgebra/Quotient.lean,Mathlib/Order/Cover.lean,Mathlib/Order/JordanHolder.lean,Mathlib/Order/KrullDimension.lean,Mathlib/Order/ListOnPartialOrderTypes.lean,Mathlib/Order/Monotone/Basic.lean,Mathlib/Order/RelSeries.lean,Mathlib/RingTheory/Artinian.lean,Mathlib/RingTheory/Finiteness.lean,Mathlib/RingTheory/Ideal/Operations.lean,Mathlib/RingTheory/Ideal/Pi.lean,Mathlib/RingTheory/KrullDimension.lean,Mathlib/RingTheory/Noetherian.lean,Mathlib/RingTheory/SimpleModule.lean,Mathlib/Topology/KrullDimension.lean,Mathlib/Topology/Sheaves/SheafCondition/EqualizerProducts.lean 24 11 ['alreadydone', 'jjaassoonn', 'leanprover-community-mathlib4-bot'] nobody
37-44431
1 month ago
469-14444
1 year ago*
0-0
0 seconds*
4979 mhk119
author:mhk119
doc(Data/Nat/Bitblast): initial commit Initial commit of Bitblast.lean where we prove equivalence of bitblast unsigned less than and bitblast addition. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data merge-conflict 202/4 Mathlib/Data/Bool/Basic.lean,Mathlib/Data/Nat/Bitwise.lean,Mathlib/Data/Nat/Pow.lean 3 49 ['ChrisHughes24', 'digama0', 'goens', 'grunweg', 'j-loreaux', 'kim-em', 'mhk119'] nobody
37-44420
1 month ago
37-44420
1 month ago
7-68358
7 days
8536 jjaassoonn
author:jjaassoonn
characteristic predicate of tensor product --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict
label:t-algebra$
399/7 Mathlib/Algebra/Category/AlgebraCat/Monoidal.lean,Mathlib/LinearAlgebra/IsTensorProduct.lean,Mathlib/LinearAlgebra/TensorProduct.lean,Mathlib/LinearAlgebra/TensorProduct/Tower.lean 4 12 ['alreadydone', 'eric-wieser', 'jjaassoonn'] nobody
37-44384
1 month ago
37-44384
1 month ago
0-0
0 seconds
11524 mcdoll
author:mcdoll
refactor: Introduce type-class for SchwartzMap --- There are a lot of other refactors to do (`seminormAux` should have a nicer name and gobble up more theorems from `seminorm`), then one can prove `integrable` and friends with only `SchwartzMapClass`. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis merge-conflict WIP 139/137 Mathlib/Analysis/Distribution/SchwartzSpace.lean,Mathlib/Analysis/Fourier/PoissonSummation.lean,Mathlib/Topology/ContinuousFunction/ZeroAtInfty.lean 3 0 [] nobody
37-44350
1 month ago
37-44350
1 month ago
0-0
0 seconds
11003 thorimur
author:thorimur
chore: migrate to `tfae` block tactic Migrates to the `tfae` block tactic syntax, eliminating uses of `tfae_have` and `tfae_finish`. --- - [ ] depends on: #11000 - [ ] depends on: #10991 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta merge-conflict blocked-by-other-PR WIP 1267/1081 Mathlib/Algebra/Exact.lean,Mathlib/Algebra/Homology/ShortComplex/ExactFunctor.lean,Mathlib/Algebra/Order/ToIntervalMod.lean,Mathlib/Analysis/BoxIntegral/Box/Basic.lean,Mathlib/Analysis/InnerProductSpace/Basic.lean,Mathlib/Analysis/LocallyConvex/WithSeminorms.lean,Mathlib/Analysis/NormedSpace/OperatorNorm/NormedSpace.lean,Mathlib/Analysis/RCLike/Basic.lean,Mathlib/Analysis/SpecificLimits/Normed.lean,Mathlib/CategoryTheory/Abelian/Exact.lean,Mathlib/CategoryTheory/Bicategory/Kan/Adjunction.lean,Mathlib/FieldTheory/Galois.lean,Mathlib/FieldTheory/KummerExtension.lean,Mathlib/GroupTheory/Nilpotent.lean,Mathlib/LinearAlgebra/Eigenspace/Zero.lean,Mathlib/MeasureTheory/Group/Action.lean,Mathlib/NumberTheory/FLT/Basic.lean,Mathlib/Order/CompactlyGenerated/Basic.lean,Mathlib/Order/Height.lean,Mathlib/Order/WellFoundedSet.lean,Mathlib/RingTheory/Bezout.lean,Mathlib/RingTheory/DiscreteValuationRing/TFAE.lean,Mathlib/RingTheory/Flat/EquationalCriterion.lean,Mathlib/RingTheory/Henselian.lean,Mathlib/RingTheory/LocalRing/RingHom/Basic.lean,Mathlib/RingTheory/Valuation/Basic.lean,Mathlib/RingTheory/Valuation/ValuationRing.lean,Mathlib/SetTheory/Ordinal/Topology.lean,Mathlib/Tactic/TFAE.lean,Mathlib/Topology/Algebra/Group/SubmonoidClosure.lean,Mathlib/Topology/Category/CompHaus/EffectiveEpi.lean,Mathlib/Topology/Category/Profinite/EffectiveEpi.lean,Mathlib/Topology/Category/Stonean/EffectiveEpi.lean,Mathlib/Topology/Inseparable.lean,Mathlib/Topology/LocallyClosed.lean,Mathlib/Topology/LocallyConstant/Basic.lean,Mathlib/Topology/NoetherianSpace.lean,Mathlib/Topology/Order/LeftRightNhds.lean,Mathlib/Topology/Separation.lean,Mathlib/Topology/UniformSpace/UniformConvergence.lean,scripts/noshake.json,test/tfae.lean 42 2 ['github-actions', 'leanprover-community-mathlib4-bot'] nobody
37-44346
1 month ago
37-44346
1 month ago
0-0
0 seconds
9819 jjaassoonn
author:jjaassoonn
fg graded ring 1. if $A$ is a noetherian graded ring, then $A_0$ is a noetherian subring of $A$ and $A$ is a finitely generated algebra over $A_0$, if $M$ is a finitely generated graded module over $A$, then each $M_n$ is a finitely generated module over $A_0$. 2. Definition of additive functions over any abelian category: if $C$ is an abelian category, a function $f : C \to \mathbb Z$ is said to be additive, if $f(y) = f(x) + f(z)$ whenever $0\to x \to y \to z \to 0$ is exact. proved some basic properties such as $f(0) = 0$ and $f(x) = f(y)$ whenever $x \cong y$ and interaction of $f$ with longer exact sequences 3. The category of finitely generated module over noetherian ring is abelian 4. A proof of Hilbert-Serre theorem: the Poincare series is actually of the form $\frac{p}{\prod(1- X^i)}$ where $p$ is polynomial The code works, but poorly written. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict WIP
label:t-algebra$
6745/217 Mathlib.lean,Mathlib/Algebra/Category/FGModuleCat/Abelian.lean,Mathlib/Algebra/Category/FGModuleCat/Basic.lean,Mathlib/Algebra/Category/FGModuleCat/EpiMono.lean,Mathlib/Algebra/Category/FGModuleCat/Kernels.lean,Mathlib/Algebra/Category/FGModuleCat/Limits.lean,Mathlib/Algebra/DirectSum/Basic.lean,Mathlib/Algebra/GradedMonoid.lean,Mathlib/Algebra/HilbertSerre/AdditiveFunction.lean,Mathlib/Algebra/HilbertSerre/FiniteInstances.lean,Mathlib/Algebra/HilbertSerre/HilbertPolynomial.lean,Mathlib/Algebra/HilbertSerre/Theorem.lean,Mathlib/Algebra/Module/GradeZeroModule.lean,Mathlib/Algebra/Module/GradedModule.lean,Mathlib/AlgebraicGeometry/ProjectiveSpectrum/Topology.lean,Mathlib/RingTheory/FiniteType.lean,Mathlib/RingTheory/Finiteness.lean,Mathlib/RingTheory/GradedAlgebra/Basic.lean,Mathlib/RingTheory/GradedAlgebra/HomogeneousIdeal.lean,Mathlib/RingTheory/GradedAlgebra/Noetherian.lean,Mathlib/RingTheory/GradedAlgebra/Radical.lean,Mathlib/RingTheory/GradedAlgebra/Subgrading.lean,Mathlib/RingTheory/Polynomial/Hilbert.lean,Mathlib/RingTheory/PowerSeries/Basic.lean,Mathlib/RingTheory/PowerSeries/WellKnown.lean 25 n/a ['FMLJohn', 'github-actions'] nobody
37-44332
1 month ago
unknown
unknown
13543 adomani
author:adomani
test: automatically undeprecate A test for `update_deprecations`. There are two files with deprecated declarations, but CI automatically fixes them, so that they pass the noisy tests (as well as passing fail-on-warning `lake build`). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-linter merge-conflict 345/4 .github/workflows/bors.yml,.github/workflows/build.yml,.github/workflows/build.yml.in,.github/workflows/build_fork.yml,Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/UpdateDeprecations.lean,Mathlib/test_depr.lean,Mathlib/test_depr_no_change.lean,lakefile.lean,scripts/update_deprecations.lean,test/UpdateDeprecations.lean 12 0 [] nobody
37-44183
1 month ago
37-44183
1 month ago
0-0
0 seconds
16186 joneugster
author:joneugster
chore: use emoji-variant-selector `\uFE0F` for emojis ✅️,❌️,💥️,🟡️ Append the emoji-variant selector `\uFE0F` to these 4 unicode symbols which should always be rendered as emojis. --- This has been done in core, so it makes sense to do the same in Mathlib. - [x] depends on: leanprover/lean4#5173 - [ ] depends on: #16215 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-linter merge-conflict awaiting-author blocked-by-other-PR 28/28 .github/workflows/lean4checker.yml,.github/workflows/nightly_detect_failure.yml,.github/workflows/update_dependencies_zulip.yml,scripts/lean-pr-testing-comments.sh,test/AssertExists.lean 5 3 ['github-actions', 'leanprover-community-mathlib4-bot', 'urkud'] nobody
37-44030
1 month ago
37-44030
1 month ago
7-61243
7 days
14932 eric-wieser
author:eric-wieser
chore: add nndist versions of lemmas --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis merge-conflict 108/1 Mathlib/Analysis/InnerProductSpace/Basic.lean,Mathlib/Geometry/Euclidean/Basic.lean 2 1 ['github-actions'] nobody
37-43996
1 month ago
37-43996
1 month ago
0-0
0 seconds
24064 kim-em
author:kim-em
chore: replace `norm_num` with `simp` where applicable Consider replacing a tactic with a (ahem) simpler alternative. Fairly neutral performance implications, just depends on whether we would like to encourage people to use `simp` where applicable. merge-conflict 345/345 Archive/Examples/MersennePrimes.lean,Archive/Imo/Imo1959Q2.lean,Archive/Imo/Imo1960Q1.lean,Archive/Imo/Imo1962Q1.lean,Archive/Imo/Imo1962Q4.lean,Archive/Imo/Imo1981Q3.lean,Archive/Imo/Imo1982Q1.lean,Archive/Imo/Imo2001Q2.lean,Archive/Imo/Imo2005Q4.lean,Archive/Imo/Imo2006Q3.lean,Archive/Imo/Imo2008Q4.lean,Archive/Imo/Imo2024Q1.lean,Archive/Imo/Imo2024Q5.lean,Archive/Imo/Imo2024Q6.lean,Archive/Wiedijk100Theorems/AbelRuffini.lean,Archive/Wiedijk100Theorems/CubingACube.lean,Archive/Wiedijk100Theorems/SumOfPrimeReciprocalsDiverges.lean,Counterexamples/Cyclotomic105.lean,Counterexamples/Phillips.lean,Mathlib/Algebra/Field/NegOnePow.lean,Mathlib/Algebra/Homology/HomotopyCategory/MappingCone.lean,Mathlib/Algebra/Order/CauSeq/BigOperators.lean,Mathlib/Algebra/Polynomial/FieldDivision.lean,Mathlib/Algebra/Polynomial/Roots.lean,Mathlib/Algebra/Polynomial/SpecificDegree.lean,Mathlib/Algebra/Ring/BooleanRing.lean,Mathlib/Algebra/Star/CHSH.lean,Mathlib/AlgebraicGeometry/EllipticCurve/IsomOfJ.lean,Mathlib/AlgebraicTopology/DoldKan/Faces.lean,Mathlib/Analysis/Analytic/Inverse.lean,Mathlib/Analysis/Asymptotics/AsymptoticEquivalent.lean,Mathlib/Analysis/BoxIntegral/UnitPartition.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Basic.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Order.lean,Mathlib/Analysis/CStarAlgebra/Module/Defs.lean,Mathlib/Analysis/Calculus/FDeriv/Measurable.lean,Mathlib/Analysis/Calculus/FDeriv/Norm.lean,Mathlib/Analysis/Calculus/FDeriv/Symmetric.lean,Mathlib/Analysis/Complex/AbelLimit.lean,Mathlib/Analysis/Convex/Between.lean,Mathlib/Analysis/Convex/Function.lean,Mathlib/Analysis/Convolution.lean,Mathlib/Analysis/Fourier/AddCircle.lean,Mathlib/Analysis/Fourier/AddCircleMulti.lean,Mathlib/Analysis/Fourier/Inversion.lean,Mathlib/Analysis/Fourier/RiemannLebesgueLemma.lean,Mathlib/Analysis/InnerProductSpace/NormPow.lean,Mathlib/Analysis/InnerProductSpace/Projection.lean,Mathlib/Analysis/InnerProductSpace/l2Space.lean,Mathlib/Analysis/MeanInequalities.lean,Mathlib/Analysis/MellinInversion.lean,Mathlib/Analysis/Normed/Affine/Simplex.lean,Mathlib/Analysis/Normed/Algebra/TrivSqZeroExt.lean,Mathlib/Analysis/Normed/Group/ControlledClosure.lean,Mathlib/Analysis/Normed/Lp/lpSpace.lean,Mathlib/Analysis/Normed/Operator/Banach.lean,Mathlib/Analysis/Normed/Ring/Units.lean,Mathlib/Analysis/NormedSpace/HahnBanach/Separation.lean,Mathlib/Analysis/NormedSpace/MStructure.lean,Mathlib/Analysis/NormedSpace/RieszLemma.lean,Mathlib/Analysis/Oscillation.lean,Mathlib/Analysis/SpecialFunctions/BinaryEntropy.lean,Mathlib/Analysis/SpecialFunctions/Complex/Log.lean,Mathlib/Analysis/SpecialFunctions/ContinuousFunctionalCalculus/Rpow/Basic.lean,Mathlib/Analysis/SpecialFunctions/ContinuousFunctionalCalculus/Rpow/Isometric.lean,Mathlib/Analysis/SpecialFunctions/ExpDeriv.lean,Mathlib/Analysis/SpecialFunctions/Gamma/Beta.lean,Mathlib/Analysis/SpecialFunctions/Gamma/BohrMollerup.lean,Mathlib/Analysis/SpecialFunctions/Gamma/Deligne.lean,Mathlib/Analysis/SpecialFunctions/Gaussian/GaussianIntegral.lean,Mathlib/Analysis/SpecialFunctions/Integrals.lean,Mathlib/Analysis/SpecialFunctions/Log/Monotone.lean,Mathlib/Analysis/SpecialFunctions/Pow/Real.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Angle.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Basic.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Complex.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Inverse.lean,Mathlib/Combinatorics/Additive/AP/Three/Behrend.lean,Mathlib/Combinatorics/Additive/SmallTripling.lean,Mathlib/Combinatorics/Extremal/RuzsaSzemeredi.lean,Mathlib/Combinatorics/SimpleGraph/Density.lean,Mathlib/Combinatorics/SimpleGraph/Regularity/Bound.lean,Mathlib/Combinatorics/SimpleGraph/Regularity/Chunk.lean,Mathlib/Combinatorics/SimpleGraph/Regularity/Increment.lean,Mathlib/Combinatorics/SimpleGraph/Regularity/Lemma.lean,Mathlib/Combinatorics/SimpleGraph/Triangle/Basic.lean,Mathlib/Combinatorics/SimpleGraph/Triangle/Counting.lean,Mathlib/Computability/Ackermann.lean,Mathlib/Computability/AkraBazzi/AkraBazzi.lean,Mathlib/Computability/DFA.lean,Mathlib/Data/Complex/Basic.lean,Mathlib/Data/Complex/Trigonometric.lean,Mathlib/Data/Nat/Bits.lean,Mathlib/Data/Nat/Choose/Central.lean,Mathlib/Data/Nat/Choose/Sum.lean,Mathlib/Data/Nat/Digits.lean,Mathlib/Data/Nat/Prime/Defs.lean,Mathlib/Data/Real/GoldenRatio.lean,Mathlib/Data/Real/Pi/Bounds.lean,Mathlib/Data/Real/Pi/Irrational.lean 171 9 ['github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'leanprover-community-mathlib4-bot'] nobody
37-5710
1 month ago
37-5711
1 month ago
11-65652
11 days
22269 Thmoas-Guan
author:Thmoas-Guan
chore(Algebra): replace Submodule.quotient.mk with Submodule.mkQ Replace Submodule.quotient.mk with Submodule.mkQ as much as possible as it have better composition property and more direct lemmas, making it more similarly with `Ideal.Quotient.mk` (except Algebra.Lie.Quotient.Basic for ones more familiar with these area) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict awaiting-author
label:t-algebra$
431/218 Mathlib/Algebra/Exact.lean,Mathlib/Algebra/Module/CharacterModule.lean,Mathlib/Algebra/Module/LocalizedModule/Submodule.lean,Mathlib/Algebra/Module/PID.lean,Mathlib/Algebra/Module/Torsion.lean,Mathlib/Algebra/Module/ZLattice/Basic.lean,Mathlib/LinearAlgebra/Dimension/Constructions.lean,Mathlib/LinearAlgebra/Dimension/RankNullity.lean,Mathlib/LinearAlgebra/Dual/Lemmas.lean,Mathlib/LinearAlgebra/Isomorphisms.lean,Mathlib/LinearAlgebra/Projection.lean,Mathlib/LinearAlgebra/Quotient/Basic.lean,Mathlib/LinearAlgebra/Quotient/Defs.lean,Mathlib/LinearAlgebra/Quotient/Pi.lean,Mathlib/LinearAlgebra/SModEq.lean,Mathlib/LinearAlgebra/Semisimple.lean,Mathlib/LinearAlgebra/TensorProduct/Quotient.lean,Mathlib/LinearAlgebra/TensorProduct/RightExactness.lean,Mathlib/NumberTheory/RamificationInertia/Basic.lean,Mathlib/RepresentationTheory/GroupCohomology/LowDegree.lean,Mathlib/RingTheory/AdicCompletion/Algebra.lean,Mathlib/RingTheory/AdicCompletion/Basic.lean,Mathlib/RingTheory/AdicCompletion/Exactness.lean,Mathlib/RingTheory/AdicCompletion/Functoriality.lean,Mathlib/RingTheory/Flat/FaithfullyFlat/Basic.lean,Mathlib/RingTheory/Ideal/Colon.lean,Mathlib/RingTheory/Ideal/Quotient/Basic.lean,Mathlib/RingTheory/Ideal/Quotient/Defs.lean,Mathlib/RingTheory/Ideal/Quotient/Operations.lean,Mathlib/RingTheory/PowerBasis.lean,Mathlib/RingTheory/QuotSMulTop.lean,Mathlib/RingTheory/Smooth/Basic.lean,Mathlib/RingTheory/TensorProduct/Quotient.lean 33 10 ['Thmoas-Guan', 'alreadydone', 'erdOne', 'github-actions', 'grunweg', 'leanprover-bot'] nobody
36-36735
1 month ago
36-36735
1 month ago
16-61571
16 days
18202 ADedecker
author:ADedecker
chore: refactor algebraic filter bases --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-topology merge-conflict
label:t-algebra$
1086/1315 Mathlib/Analysis/Distribution/SchwartzSpace.lean,Mathlib/Analysis/LocallyConvex/AbsConvex.lean,Mathlib/Analysis/LocallyConvex/Barrelled.lean,Mathlib/Analysis/LocallyConvex/WeakDual.lean,Mathlib/Analysis/LocallyConvex/WithSeminorms.lean,Mathlib/Analysis/Normed/Operator/WeakOperatorTopology.lean,Mathlib/FieldTheory/KrullTopology.lean,Mathlib/RingTheory/DedekindDomain/FiniteAdeleRing.lean,Mathlib/Topology/Algebra/FilterBasis.lean,Mathlib/Topology/Algebra/Module/UniformConvergence.lean,Mathlib/Topology/Algebra/Nonarchimedean/AdicTopology.lean,Mathlib/Topology/Algebra/Nonarchimedean/Bases.lean,Mathlib/Topology/Algebra/UniformFilterBasis.lean,Mathlib/Topology/Algebra/Valued/ValuationTopology.lean 14 1 ['github-actions'] nobody
36-36667
1 month ago
36-36667
1 month ago
0-0
0 seconds
23546 JovanGerb
author:JovanGerb
feat(LinearAlgebra/AffineSpace/AffineSubspace): rename `AffineSubspace.mk'` to `Submodule.shift` In addition to renaming, I've refactored the code a bit: - `mem_mk'_iff_vsub_mem` was obsolete since it was the same as `mem_mk'`, so I removed it (this is due to a change in the definition I made recently) - I added a nonempty instance for `shift` - I added a simp lemma that `shift` isn't equal to `⊥` (the empty affine subspace). I need this for the next point. - Edit: I'll leave this for a later PR. ~I proved a simp lemma that a `shift` is parallel to a `shift` if and only if the linear subspaces are the same.~ - I renamed `mk'_eq` to `shift_direction_eq_self `. - I renamed `eq_or_eq_secondInter_of_mem_mk'_span_singleton_iff_mem` to `eq_or_eq_secondInter_iff_mem_of_mem_shift_span_singleton`. I think it is better to put the `of_mem_mk'_span_singleton` at the end of the name. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-euclidean-geometry merge-conflict 128/99 Mathlib/Algebra/Module/ZLattice/Basic.lean,Mathlib/Geometry/Euclidean/Basic.lean,Mathlib/Geometry/Euclidean/MongePoint.lean,Mathlib/Geometry/Euclidean/PerpBisector.lean,Mathlib/Geometry/Euclidean/Sphere/SecondInter.lean,Mathlib/Geometry/Euclidean/Sphere/Tangent.lean,Mathlib/LinearAlgebra/AffineSpace/AffineSubspace/Defs.lean 7 4 ['JovanGerb', 'github-actions', 'leanprover-community-bot-assistant'] nobody
36-19167
1 month ago
36-19168
1 month ago
26-25420
26 days
24483 Parcly-Taxel
author:Parcly-Taxel
chore: delete >6 month old deprecations (2024-10) See #24271 for the general pattern of regex used in the first (automated) commit. The date range used in this PR is `2024-10-..`. tech debt merge-conflict 2/1182 Mathlib/Algebra/BigOperators/Group/List/Basic.lean,Mathlib/Algebra/CharP/Two.lean,Mathlib/Algebra/Order/Monoid/Unbundled/WithTop.lean,Mathlib/AlgebraicGeometry/Morphisms/ClosedImmersion.lean,Mathlib/AlgebraicGeometry/Morphisms/Preimmersion.lean,Mathlib/AlgebraicGeometry/Restrict.lean,Mathlib/Analysis/Analytic/Basic.lean,Mathlib/Analysis/Calculus/ContDiff/Basic.lean,Mathlib/Analysis/Calculus/ContDiff/Defs.lean,Mathlib/Analysis/Calculus/Deriv/Basic.lean,Mathlib/Analysis/Calculus/Deriv/Comp.lean,Mathlib/Analysis/Calculus/FDeriv/Basic.lean,Mathlib/Analysis/Calculus/FDeriv/Comp.lean,Mathlib/Analysis/Calculus/LineDeriv/Basic.lean,Mathlib/Analysis/Complex/ReImTopology.lean,Mathlib/Analysis/Complex/UpperHalfPlane/Topology.lean,Mathlib/Analysis/LocallyConvex/WeakOperatorTopology.lean,Mathlib/Analysis/LocallyConvex/WithSeminorms.lean,Mathlib/Analysis/Normed/Operator/Banach.lean,Mathlib/Analysis/Normed/Operator/LinearIsometry.lean,Mathlib/Analysis/NormedSpace/OperatorNorm/NormedSpace.lean,Mathlib/CategoryTheory/Limits/Preserves/Limits.lean,Mathlib/CategoryTheory/Sites/Canonical.lean,Mathlib/Data/ENNReal/Inv.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/Data/List/Flatten.lean,Mathlib/Data/List/SplitBy.lean,Mathlib/Data/Nat/Factorization/Basic.lean,Mathlib/Data/Nat/Factorization/Defs.lean,Mathlib/Data/Nat/Factorization/PrimePow.lean,Mathlib/Data/Set/Subset.lean,Mathlib/FieldTheory/IntermediateField/Adjoin/Algebra.lean,Mathlib/Geometry/Manifold/ContMDiff/Defs.lean,Mathlib/Geometry/Manifold/LocalInvariantProperties.lean,Mathlib/Geometry/Manifold/MFDeriv/Basic.lean,Mathlib/GroupTheory/CosetCover.lean,Mathlib/GroupTheory/GroupAction/Blocks.lean,Mathlib/LinearAlgebra/Eigenspace/Basic.lean,Mathlib/MeasureTheory/Constructions/BorelSpace/Basic.lean,Mathlib/MeasureTheory/Function/StronglyMeasurable/AEStronglyMeasurable.lean,Mathlib/MeasureTheory/Measure/DiracProba.lean,Mathlib/MeasureTheory/Measure/FiniteMeasure.lean,Mathlib/MeasureTheory/Measure/ProbabilityMeasure.lean,Mathlib/NumberTheory/NumberField/Embeddings.lean,Mathlib/Order/InitialSeg.lean,Mathlib/Order/WellFounded.lean,Mathlib/Probability/Density.lean,Mathlib/RingTheory/Finiteness/Cardinality.lean,Mathlib/RingTheory/Finiteness/Ideal.lean,Mathlib/RingTheory/Jacobson/Ring.lean,Mathlib/RingTheory/Localization/Cardinality.lean,Mathlib/RingTheory/PowerSeries/Basic.lean,Mathlib/RingTheory/Spectrum/Prime/TensorProduct.lean,Mathlib/RingTheory/Spectrum/Prime/Topology.lean,Mathlib/SetTheory/Game/Nim.lean,Mathlib/SetTheory/PGame/Algebra.lean,Mathlib/Tactic/FunProp/ContDiff.lean,Mathlib/Topology/AlexandrovDiscrete.lean,Mathlib/Topology/Algebra/ConstMulAction.lean,Mathlib/Topology/Algebra/Constructions.lean,Mathlib/Topology/Algebra/Constructions/DomMulAct.lean,Mathlib/Topology/Algebra/Group/Basic.lean,Mathlib/Topology/Algebra/Group/CompactOpen.lean,Mathlib/Topology/Algebra/Group/Quotient.lean,Mathlib/Topology/Algebra/GroupWithZero.lean,Mathlib/Topology/Algebra/InfiniteSum/Basic.lean,Mathlib/Topology/Algebra/Module/Alternating/Topology.lean,Mathlib/Topology/Algebra/Module/Equiv.lean,Mathlib/Topology/Algebra/Module/Multilinear/Topology.lean,Mathlib/Topology/Algebra/Module/StrongTopology.lean,Mathlib/Topology/Algebra/Module/WeakBilin.lean,Mathlib/Topology/Algebra/Monoid.lean,Mathlib/Topology/Algebra/MulAction.lean,Mathlib/Topology/Algebra/Ring/Ideal.lean,Mathlib/Topology/Algebra/SeparationQuotient/Section.lean,Mathlib/Topology/Algebra/StarSubalgebra.lean,Mathlib/Topology/Bases.lean,Mathlib/Topology/Category/Profinite/Nobeling/Induction.lean,Mathlib/Topology/Category/TopCat/EffectiveEpi.lean,Mathlib/Topology/Category/TopCat/Limits/Products.lean,Mathlib/Topology/Category/TopCat/Limits/Pullbacks.lean,Mathlib/Topology/Clopen.lean,Mathlib/Topology/CompactOpen.lean,Mathlib/Topology/Compactness/Compact.lean,Mathlib/Topology/Compactness/Lindelof.lean,Mathlib/Topology/Compactness/LocallyCompact.lean,Mathlib/Topology/Compactness/SigmaCompact.lean,Mathlib/Topology/Connected/Basic.lean,Mathlib/Topology/Connected/Clopen.lean,Mathlib/Topology/Connected/PathConnected.lean,Mathlib/Topology/Connected/TotallyDisconnected.lean,Mathlib/Topology/Constructions.lean,Mathlib/Topology/Constructions/SumProd.lean,Mathlib/Topology/ContinuousMap/Bounded/Basic.lean,Mathlib/Topology/ContinuousMap/ContinuousMapZero.lean,Mathlib/Topology/ContinuousMap/Sigma.lean,Mathlib/Topology/ContinuousMap/T0Sierpinski.lean,Mathlib/Topology/ContinuousOn.lean,Mathlib/Topology/Covering.lean,Mathlib/Topology/Defs/Induced.lean 139 3 ['github-actions', 'leanprover-community-bot-assistant'] nobody
35-41124
1 month ago
35-41126
1 month ago
4-54091
4 days
23953 b-reinke
author:b-reinke
feat(Data/Matroid/Tutte): define the Tutte polynomial of a matroid This PR defines the Tutte polynomial of a matroid and shows basic properties. - [ ] depends on: #23926 - [ ] depends on #24336 - [ ] depends on: #23951 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data merge-conflict blocked-by-other-PR WIP 111/0 Mathlib/Algebra/BigOperators/Finprod.lean,Mathlib/Data/Matroid/Tutte/Basic.lean,Mathlib/Data/Set/Image.lean 3 7 ['apnelson1', 'b-reinke', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
35-19763
1 month ago
37-45416
1 month ago
0-0
0 seconds
23590 mariainesdff
author:mariainesdff
feat(RingTheory/Valuation/Extension): add algebra instances Provide algebra instances for valuation subrings and residue fields. Co-authored-by: @faenuccio --- - [ ] depends on: #23408 - [ ] depends on: #23584 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict
label:t-algebra$
88/19 Mathlib.lean,Mathlib/RingTheory/Valuation/Extension.lean,Mathlib/RingTheory/Valuation/Integers.lean,Mathlib/RingTheory/Valuation/ValuationSubring.lean 4 19 ['github-actions', 'jjdishere', 'leanprover-community-bot-assistant', 'mariainesdff', 'mathlib4-dependent-issues-bot'] nobody
35-18628
1 month ago
35-18629
1 month ago
0-1121
18 minutes
21853 smmercuri
author:smmercuri
feat: the adele ring of a number field is locally compact --- - [ ] depends on: #21158 - [ ] depends on: #21847 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-number-theory merge-conflict blocked-by-other-PR WIP 398/3 Mathlib.lean,Mathlib/Algebra/Order/GroupWithZero/Canonical.lean,Mathlib/NumberTheory/NumberField/AdeleRing.lean,Mathlib/RingTheory/DedekindDomain/AdicValuation.lean,Mathlib/RingTheory/DedekindDomain/FiniteAdeleRing.lean,Mathlib/RingTheory/Ideal/Quotient/Basic.lean,Mathlib/Topology/Algebra/Group/Basic.lean,Mathlib/Topology/Algebra/Valued/LocallyCompact.lean,Mathlib/Topology/Algebra/Valued/WithZeroMulInt.lean 9 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
35-9767
1 month ago
37-45168
1 month ago
0-0
0 seconds
15654 TpmKranz
author:TpmKranz
feat(Computability): language-preserving maps between NFA and RE Map REs to NFAs via Thompson's construction and NFAs to REs using GNFAs Last chunk of #12648 --- - [ ] depends on: #15651 - [ ] depends on: #15649 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-zulip t-computability new-contributor merge-conflict blocked-by-other-PR 985/2 Mathlib.lean,Mathlib/Computability/GNFA.lean,Mathlib/Computability/Language.lean,Mathlib/Computability/NFA.lean,Mathlib/Computability/RegularExpressions.lean,Mathlib/Data/FinEnum/Option.lean,docs/references.bib 7 3 ['github-actions', 'leanprover-community-mathlib4-bot', 'meithecatte'] nobody
34-77865
1 month ago
34-77870
1 month ago
0-179
2 minutes
19315 quangvdao
author:quangvdao
feat(Data/Finsupp/Fin): Add `Finsupp` operations on `Fin` tuple This PR adds more analogues of operations on `Fin` tuples to the `Finsupp` setting. Before, there were only `Finsupp.cons` and `Finsupp.tail`. Now there are also `Finsupp.snoc`, `Finsupp.insertNth`, `Finsupp.init`, and `Finsupp.removeNth`. These all come with supporting lemmas. I also removed the porting comment about `succAboveCases` in `Data/Fin/Basic`, and added a lemma about `succAbove` in `Data/Fin/Tuple/Basic`. --- - [x] depends on: #20361 - [x] depends on: #20771 - [x] depends on: #20770 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data merge-conflict awaiting-author 193/16 Mathlib/Algebra/BigOperators/Fin.lean,Mathlib/Algebra/BigOperators/Finsupp.lean,Mathlib/Algebra/MvPolynomial/Equiv.lean,Mathlib/Data/Finsupp/Fin.lean,Mathlib/RingTheory/MvPolynomial/Homogeneous.lean,scripts/nolints_prime_decls.txt 6 44 ['YaelDillies', 'github-actions', 'j-loreaux', 'kbuzzard', 'mathlib4-dependent-issues-bot', 'quangvdao'] nobody
33-79826
1 month ago
33-79826
1 month ago
43-81255
43 days
21751 vihdzp
author:vihdzp
refactor(SetTheory/Ordinal/Arithmetic): rework `Ordinal.pred` API This PR does the following: - give a simpler definition of `Ordinal.pred` - replace `¬ ∃ a, o = succ a` and `∀ a, o ≠ succ a` by `IsSuccPrelimit o` throughout - improve theorem names --- There's a legitimate question of whether we even want `Ordinal.pred` (see [Zulip](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Ordinal.2Epred)) but this should be a good change in the meanwhile regardless. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-set-theory maintainer-merge merge-conflict 102/67 Mathlib/SetTheory/Ordinal/Arithmetic.lean,Mathlib/SetTheory/Ordinal/Exponential.lean 2 13 ['YaelDillies', 'github-actions', 'grunweg', 'vihdzp'] nobody
33-79798
1 month ago
80-58425
2 months ago
36-50134
36 days
19464 adomani
author:adomani
test: removed merge-conflict --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) CI merge-conflict delegated WIP 22/1 .github/workflows/PR_summary.yml,scripts/zulip_emoji_merge_delegate.py 2 10 ['adomani', 'github-actions', 'leanprover-community-bot-assistant'] nobody
33-4750
1 month ago
33-4752
1 month ago
0-0
0 seconds
7907 urkud
author:urkud
feat: introduce `NthRoot` notation class Also use it for `Real.sqrt`, and replace the few occurrences of `sqrt` that do not already use the notation. --- [Zulip](https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/.60Sqrt.60.20notation.20typeclass/near/400086502) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-analysis awaiting-CI merge-conflict
label:t-algebra$
193/156 Archive/Imo/Imo1959Q2.lean,Archive/Imo/Imo1960Q2.lean,Archive/Imo/Imo2001Q2.lean,Archive/Imo/Imo2006Q3.lean,Archive/Imo/Imo2008Q3.lean,Archive/Imo/Imo2008Q4.lean,Archive/Sensitivity.lean,Archive/Wiedijk100Theorems/AreaOfACircle.lean,Mathlib.lean,Mathlib/Algebra/NthRoot.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Instances.lean,Mathlib/Analysis/Complex/AbelLimit.lean,Mathlib/Analysis/RCLike/Basic.lean,Mathlib/Analysis/SpecialFunctions/Pow/Asymptotics.lean,Mathlib/Analysis/SpecialFunctions/Pow/Real.lean,Mathlib/Analysis/SpecialFunctions/Stirling.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Basic.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Bounds.lean,Mathlib/Data/Real/GoldenRatio.lean,Mathlib/Data/Real/Sqrt.lean,Mathlib/LinearAlgebra/Matrix/PosDef.lean,Mathlib/MeasureTheory/Measure/Lebesgue/VolumeOfBalls.lean,Mathlib/NumberTheory/Harmonic/GammaDeriv.lean,Mathlib/NumberTheory/NumberField/CanonicalEmbedding/ConvexBody.lean,Mathlib/NumberTheory/NumberField/ClassNumber.lean,Mathlib/NumberTheory/NumberField/Discriminant/Basic.lean,Mathlib/Probability/Distributions/Gaussian.lean,MathlibTest/positivity.lean 28 9 ['eric-wieser', 'github-actions', 'kmill', 'urkud'] nobody
32-20540
1 month ago
286-34098
9 months ago
0-0
0 seconds
9273 grunweg
author:grunweg
feat: extended charts are local diffeomorphisms on their source --- TODO: I think this should hold at any interior point - as the inverse of the extended chart, restricted to the interior of its source, will be a local inverse. The analogous result for un-extended charts is shown in #8160. Unresolved questions - are all the tiny API lemmas useful; are any more missing? - do I want similar results for `extChartAt`? (In any case, they are easy to deduce.) - [ ] depends on: #8738 for simplicity [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-differential-geometry merge-conflict 225/12 Mathlib/Geometry/Manifold/ContMDiff/Atlas.lean,Mathlib/Geometry/Manifold/LocalDiffeomorph.lean,Mathlib/Topology/Algebra/Module/Basic.lean 3 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
31-80975
1 month ago
unknown
unknown
23040 grunweg
author:grunweg
feat: define immersions and smooth embeddings in infinite dimensions Sadly, we cannot prove most nice things about them yet, as we don't have the inverse function theorem yet. TODO: prove the few things we can already say --- - [ ] depends on: #23175 (preliminaries) - [ ] depends on: #23186 - [ ] depends on: another PR, about `MSplitAt` (to be filed) - and perhaps some prerequisites about products of complemented modules etc. - [ ] depends on: #23219 (preliminaries about local diffeomorphisms) - [ ] depends on: #8738 - in fact, #9273 is not a strict pre-requisite for this. It suffices to know "extended charts have invertible differentials", which [isInvertible_mfderiv_extChartAt](https://leanprover-community.github.io/mathlib4_docs/Mathlib/Geometry/Manifold/MFDeriv/Atlas.html#isInvertible_mfderiv_extChartAt) mostly proves. (There's nothing wrong with completing that PR, for all interior points.) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-differential-geometry merge-conflict blocked-by-other-PR WIP 967/0 Mathlib.lean,Mathlib/Analysis/NormedSpace/HahnBanach/Splits.lean,Mathlib/Geometry/Manifold/IsImmersionEmbedding.lean,Mathlib/Geometry/Manifold/LocalDiffeomorph.lean,Mathlib/Geometry/Manifold/MSplits.lean 5 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
31-75190
1 month ago
31-78717
1 month ago
0-0
0 seconds
24550 grunweg
author:grunweg
feat: define `SliceModel` typeclass for models with corners for embedded submanifolds Still work in progress: TODO write a proper module doc-string and commit message. --- - [ ] depends on: #23040 (at least morally) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-differential-geometry merge-conflict blocked-by-other-PR WIP 1214/0 Mathlib.lean,Mathlib/Analysis/NormedSpace/HahnBanach/Splits.lean,Mathlib/Geometry/Manifold/IsImmersionEmbedding.lean,Mathlib/Geometry/Manifold/LocalDiffeomorph.lean,Mathlib/Geometry/Manifold/MSplits.lean,Mathlib/Geometry/Manifold/SliceModel.lean 6 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
31-75128
1 month ago
31-75560
1 month ago
0-0
0 seconds
19985 vihdzp
author:vihdzp
feat(SetTheory/ZFC/Ordinal): Lean ordinals to ZFC ordinals We define `Ordinal.toZFSet` and prove that its outputs are precisely the ZFC ordinals. --- - [ ] depends on: #19946 - [x] depends on: #19970 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-set-theory merge-conflict 208/6 Mathlib/Order/SuccPred/CompleteLinearOrder.lean,Mathlib/SetTheory/ZFC/Basic.lean,Mathlib/SetTheory/ZFC/Ordinal.lean,Mathlib/SetTheory/ZFC/Rank.lean 4 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
31-13249
1 month ago
31-13252
1 month ago
0-562
9 minutes
17027 vihdzp
author:vihdzp
feat(SetTheory/ZFC/Ordinal): von Neumann hierarchy of sets --- - [x] depends on: #16996 - [x] depends on: #17016 - [x] depends on: #17026 - [x] depends on: #18239 - [ ] depends on: #19946 - [x] depends on: #19967 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-set-theory merge-conflict 204/29 Mathlib.lean,Mathlib/SetTheory/Ordinal/Basic.lean,Mathlib/SetTheory/ZFC/Basic.lean,Mathlib/SetTheory/ZFC/Neumann.lean,Mathlib/SetTheory/ZFC/Rank.lean 5 8 ['alreadydone', 'github-actions', 'mathlib4-dependent-issues-bot', 'vihdzp'] nobody
31-13200
1 month ago
31-13202
1 month ago
0-344
5 minutes
18755 FR-vdash-bot
author:FR-vdash-bot
refactor: deprecate `LinearIsometryClass` --- - [ ] depends on: #18748 - [ ] depends on: #18754 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-analysis merge-conflict blocked-by-other-PR
label:t-algebra$
243/116 Mathlib/Analysis/CStarAlgebra/Spectrum.lean,Mathlib/Analysis/LocallyConvex/WeakOperatorTopology.lean,Mathlib/Analysis/Normed/Algebra/Spectrum.lean,Mathlib/Analysis/Normed/Group/Uniform.lean,Mathlib/Analysis/Normed/Operator/LinearIsometry.lean,Mathlib/Topology/Algebra/Module/Basic.lean,Mathlib/Topology/Algebra/Module/CharacterSpace.lean,Mathlib/Topology/Algebra/Module/FiniteDimension.lean,Mathlib/Topology/Algebra/Module/StrongTopology.lean,Mathlib/Topology/Algebra/Module/WeakDual.lean,Mathlib/Topology/Homeomorph.lean,Mathlib/Topology/MetricSpace/Isometry.lean,scripts/no_lints_prime_decls.txt 13 5 ['FR-vdash-bot', 'github-actions', 'leanprover-bot', 'mathlib4-dependent-issues-bot'] nobody
30-84574
30 days ago
206-40835
6 months ago
0-602
10 minutes
24248 urkud
author:urkud
feat(HaarToSphere): add integrability lemmas --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-measure-probability merge-conflict 99/6 Mathlib/MeasureTheory/Constructions/HaarToSphere.lean,Mathlib/MeasureTheory/Integral/Prod.lean 2 2 ['github-actions', 'leanprover-community-bot-assistant'] nobody
29-45005
29 days ago
29-45007
29 days ago
0-0
0 seconds
24523 dagurtomas
author:dagurtomas
feat(Condensed): closed symmetric monoidal structure on light condensed modules --- - [ ] depends on: #24485 - [ ] depends on: #24490 - [ ] depends on: #24522 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-condensed merge-conflict blocked-by-other-PR WIP 473/2 Mathlib.lean,Mathlib/CategoryTheory/Localization/Monoidal/Basic.lean,Mathlib/CategoryTheory/Localization/Monoidal/Braided.lean,Mathlib/CategoryTheory/Monoidal/Braided/Basic.lean,Mathlib/CategoryTheory/Monoidal/Braided/Transport.lean,Mathlib/CategoryTheory/Sites/Monoidal.lean,Mathlib/Condensed/Light/Monoidal.lean,Mathlib/Condensed/Light/Small.lean 8 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
29-31270
29 days ago
29-31271
29 days ago
0-133
2 minutes
24019 urkud
author:urkud
feat(Analysis): Poincaré lemma for 1-forms --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis merge-conflict 704/33 Mathlib.lean,Mathlib/Analysis/Calculus/ContDiff/Basic.lean,Mathlib/Analysis/Calculus/Deriv/Basic.lean,Mathlib/Analysis/Calculus/Deriv/CompMul.lean,Mathlib/Analysis/Calculus/Deriv/Shift.lean,Mathlib/Analysis/Calculus/FDeriv/Analytic.lean,Mathlib/Analysis/Calculus/FDeriv/Basic.lean,Mathlib/Analysis/Calculus/FDeriv/Equiv.lean,Mathlib/Analysis/Calculus/Gradient/Basic.lean,Mathlib/Analysis/Calculus/Poincare/OneForm.lean,Mathlib/Analysis/Calculus/TangentCone.lean,Mathlib/MeasureTheory/Integral/DivergenceTheorem.lean,Mathlib/MeasureTheory/Integral/PathIntegral/Basic.lean,Mathlib/Topology/Homotopy/Path.lean,Mathlib/Topology/Path.lean,Mathlib/Topology/UnitInterval.lean 16 4 ['github-actions', 'leanprover-community-bot-assistant'] nobody
29-4114
29 days ago
29-4116
29 days ago
0-0
0 seconds
24477 mariainesdff
author:mariainesdff
feat(RingTheory/Ideal/Span): subideals form a complete lattice Co-authored-by: @AntoineChambert-Loir --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict awaiting-author
label:t-algebra$
33/0 Mathlib/RingTheory/Ideal/Span.lean 1 8 ['alreadydone', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'mariainesdff'] nobody
28-83301
28 days ago
28-83301
28 days ago
9-2345
9 days
24642 grunweg
author:grunweg
WIP-feat: add layercake formula for ENNReal-valued functions Not much to see here yet; some significant amount of work remains. --- - [ ] depends on: #24643 - [ ] depends on: #24640 (based on that PR for simplicity) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) carleson t-analysis merge-conflict WIP 189/24 Mathlib/Analysis/SpecialFunctions/Pow/Integral.lean,Mathlib/MeasureTheory/Function/LpSeminorm/Basic.lean,Mathlib/MeasureTheory/Function/LpSpace/Basic.lean,Mathlib/MeasureTheory/Integral/Layercake.lean 4 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
28-13425
28 days ago
28-13428
28 days ago
0-0
0 seconds
21712 grunweg
author:grunweg
chore: generalise more lemmas to `ContinuousENorm` --- - [x] depends on: #21781 (minor drive-by clean-up) - [x] depends on: #21670 - [x] depends on: #22708 (extracted from this) - some parts depend on #21433 (or better: #22175); when the dependent PR has landed, I will re-assess whether to split these into a separate PR [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) carleson t-measure-probability awaiting-CI merge-conflict 76/31 Mathlib/Analysis/Normed/MulAction.lean,Mathlib/MeasureTheory/Function/LpSeminorm/Basic.lean,Mathlib/MeasureTheory/Function/LpSpace/Basic.lean,Mathlib/MeasureTheory/Function/LpSpace/ContinuousFunctions.lean 4 5 ['github-actions', 'grunweg', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
27-35109
27 days ago
37-45143
1 month ago
0-0
0 seconds
21375 grunweg
author:grunweg
WIP: generalise lemmas to ENorm This work is part of (and a necessary pre-requisite for) the Carleson project. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) carleson t-measure-probability awaiting-CI merge-conflict WIP 471/221 Mathlib/Analysis/NormedSpace/IndicatorFunction.lean,Mathlib/MeasureTheory/Function/L2Space.lean,Mathlib/MeasureTheory/Function/LocallyIntegrable.lean,Mathlib/MeasureTheory/Function/LpOrder.lean,Mathlib/MeasureTheory/Function/LpSeminorm/Basic.lean,Mathlib/MeasureTheory/Function/LpSeminorm/ChebyshevMarkov.lean,Mathlib/MeasureTheory/Function/LpSeminorm/CompareExp.lean,Mathlib/MeasureTheory/Function/LpSeminorm/TriangleInequality.lean,Mathlib/MeasureTheory/Function/LpSeminorm/Trim.lean,Mathlib/MeasureTheory/Function/LpSpace.lean,Mathlib/MeasureTheory/Function/SimpleFuncDenseLp.lean,Mathlib/MeasureTheory/Function/UniformIntegrable.lean,Mathlib/Probability/Independence/Integrable.lean 13 2 ['fpvandoorn', 'grunweg'] nobody
27-29484
27 days ago
37-45138
1 month ago
0-0
0 seconds
24378 urkud
author:urkud
feat(Algebra/Order/Field/Basic): generalize lemmas ... from linear ordered semifields to (commutative) groups with zero. --- I'm going to do another round of generalizing today or tomorrow, so making it a draft PR for now. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict
label:t-algebra$
183/181 Archive/OxfordInvariants/Summer2021/Week3P1.lean,Mathlib/Algebra/Order/Field/Basic.lean,Mathlib/Algebra/Order/Floor/Ring.lean,Mathlib/Algebra/Order/Floor/Semiring.lean,Mathlib/Algebra/Order/GroupWithZero/Unbundled/Basic.lean,Mathlib/Analysis/Analytic/Basic.lean,Mathlib/Analysis/Asymptotics/Lemmas.lean,Mathlib/Analysis/CStarAlgebra/ApproximateUnit.lean,Mathlib/Analysis/Calculus/BumpFunction/Basic.lean,Mathlib/Analysis/Calculus/BumpFunction/FiniteDimension.lean,Mathlib/Analysis/Calculus/BumpFunction/InnerProduct.lean,Mathlib/Analysis/Complex/AbelLimit.lean,Mathlib/Analysis/Complex/Hadamard.lean,Mathlib/Analysis/Convex/Segment.lean,Mathlib/Analysis/Convex/SpecificFunctions/Basic.lean,Mathlib/Analysis/Convex/SpecificFunctions/Pow.lean,Mathlib/Analysis/Convex/StrictConvexSpace.lean,Mathlib/Analysis/Convex/Uniform.lean,Mathlib/Analysis/Convex/Visible.lean,Mathlib/Analysis/Fourier/RiemannLebesgueLemma.lean,Mathlib/Analysis/FunctionalSpaces/SobolevInequality.lean,Mathlib/Analysis/MeanInequalitiesPow.lean,Mathlib/Analysis/Normed/Field/Lemmas.lean,Mathlib/Analysis/Normed/Field/Ultra.lean,Mathlib/Analysis/Normed/Unbundled/SmoothingSeminorm.lean,Mathlib/Analysis/NormedSpace/HomeomorphBall.lean,Mathlib/Analysis/NormedSpace/OperatorNorm/NormedSpace.lean,Mathlib/Analysis/NormedSpace/Pointwise.lean,Mathlib/Analysis/SpecialFunctions/Complex/Arg.lean,Mathlib/Analysis/SpecialFunctions/Gamma/Beta.lean,Mathlib/Analysis/SpecialFunctions/Log/Deriv.lean,Mathlib/Analysis/SpecialFunctions/MulExpNegMulSqIntegral.lean,Mathlib/Analysis/SpecialFunctions/SmoothTransition.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Bounds.lean,Mathlib/Analysis/SpecificLimits/Basic.lean,Mathlib/Analysis/SpecificLimits/FloorPow.lean,Mathlib/Analysis/SpecificLimits/Normed.lean,Mathlib/Combinatorics/Additive/AP/Three/Behrend.lean,Mathlib/Combinatorics/Schnirelmann.lean,Mathlib/Combinatorics/SimpleGraph/Regularity/Chunk.lean,Mathlib/Computability/AkraBazzi/AkraBazzi.lean,Mathlib/Computability/AkraBazzi/GrowsPolynomially.lean,Mathlib/Data/Nat/Cast/Order/Field.lean,Mathlib/Data/Real/Archimedean.lean,Mathlib/Data/Real/Cardinality.lean,Mathlib/Data/Real/Pi/Wallis.lean,Mathlib/Geometry/Euclidean/Angle/Unoriented/Affine.lean,Mathlib/Geometry/Euclidean/Angle/Unoriented/RightAngle.lean,Mathlib/Geometry/Euclidean/Sphere/Tangent.lean,Mathlib/MeasureTheory/Function/StronglyMeasurable/Basic.lean,Mathlib/MeasureTheory/Function/UniformIntegrable.lean,Mathlib/MeasureTheory/Integral/CircleIntegral.lean,Mathlib/MeasureTheory/Integral/MeanInequalities.lean,Mathlib/MeasureTheory/Integral/PeakFunction.lean,Mathlib/MeasureTheory/Measure/SeparableMeasure.lean,Mathlib/NumberTheory/Bertrand.lean,Mathlib/NumberTheory/ClassNumber/AdmissibleAbs.lean,Mathlib/NumberTheory/DiophantineApproximation/Basic.lean,Mathlib/NumberTheory/LSeries/Injectivity.lean,Mathlib/NumberTheory/LSeries/ZMod.lean,Mathlib/NumberTheory/NumberField/Discriminant/Basic.lean,Mathlib/NumberTheory/Padics/Hensel.lean,Mathlib/NumberTheory/Padics/MahlerBasis.lean,Mathlib/NumberTheory/Pell.lean,Mathlib/NumberTheory/Transcendental/Liouville/LiouvilleNumber.lean,Mathlib/Order/Filter/AtTopBot/Floor.lean,Mathlib/Order/Interval/Set/IsoIoo.lean,Mathlib/Probability/StrongLaw.lean,Mathlib/RingTheory/Perfection.lean,Mathlib/Topology/ContinuousMap/Polynomial.lean,Mathlib/Topology/Instances/AddCircle.lean,Mathlib/Topology/UrysohnsLemma.lean 72 3 ['github-actions', 'leanprover-community-bot-assistant'] nobody
27-13814
27 days ago
27-13816
27 days ago
0-0
0 seconds
21847 smmercuri
author:smmercuri
feat: `v.adicCompletionIntegers K` is compact --- - [ ] depends on: #21844 - [ ] depends on: #24872 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-number-theory merge-conflict blocked-by-other-PR WIP 459/4 Mathlib.lean,Mathlib/Algebra/Order/GroupWithZero/Canonical.lean,Mathlib/NumberTheory/NumberField/AdeleRing.lean,Mathlib/RingTheory/DedekindDomain/AdicValuation.lean,Mathlib/RingTheory/DedekindDomain/FiniteAdeleRing.lean,Mathlib/RingTheory/Ideal/Quotient/Basic.lean,Mathlib/Topology/Algebra/Group/Basic.lean,Mathlib/Topology/Algebra/UniformRing.lean,Mathlib/Topology/Algebra/Valued/LocallyCompact.lean,Mathlib/Topology/Algebra/Valued/ValuationTopology.lean,Mathlib/Topology/Algebra/Valued/WithZeroMulInt.lean 11 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
26-47640
26 days ago
37-45159
1 month ago
0-0
0 seconds
23338 WilliamCoram
author:WilliamCoram
feat: restricted power series form a ring We define restricted powerseries over a normed ring R, and show they form a ring when R has the ultrametric property. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-number-theory merge-conflict 186/0 Mathlib.lean,Mathlib/RingTheory/PowerSeries/Restricted.lean 2 18 ['Paul-Lez', 'WilliamCoram', 'github-actions', 'grunweg', 'leanprover-community-bot-assistant'] nobody
26-33783
26 days ago
26-33785
26 days ago
48-76736
48 days
24853 smmercuri
author:smmercuri
feat: dimensions of completions at infinite place extensions Let `L / K` be an extension of number fields. For a fixed `v : InfinitePlace K`, we consider the infinite places `w` of `L` that extend `v`. The main results of this PR are: - `InfinitePlace.sum_ramificationIdx_eq`: the sum over all `w` extending `v` of the ramification indices of `w` over `K` is `[K : L]`. - `InfinitePlace.finrank_eq_ramificationIdx`: the `v.Completion`-dimension of `w.Completion` equals the ramification index of `w` over `K`. --- - [ ] depends on: #24870 - [ ] depends on: #24872 - [ ] depends on: #24873 - [ ] depends on: #24875 - [ ] depends on: #24877 - [x] depends on: #24879 - [ ] depends on: #24881 - [ ] depends on: #24882 - [ ] depends on: #24884 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import FLT merge-conflict blocked-by-other-PR 918/1 Mathlib.lean,Mathlib/Analysis/Normed/Field/WithAbs.lean,Mathlib/Data/Subtype.lean,Mathlib/NumberTheory/NumberField/InfinitePlace/Basic.lean,Mathlib/NumberTheory/NumberField/InfinitePlace/Dimension.lean,Mathlib/NumberTheory/NumberField/InfinitePlace/Embeddings.lean,Mathlib/NumberTheory/NumberField/InfinitePlace/Ramification.lean,Mathlib/Topology/Algebra/UniformRing.lean 8 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
26-16899
26 days ago
26-16901
26 days ago
0-1
1 second
4197 joelriou
author:joelriou
feat/refactor: redefinition of homology + derived categories This PR contains a redefinition of homology, theorems about localization of categories, including triangulated categories, a construction of the derived category of an abelian category, derived functors, spectral sequences, etc. (This is made a PR only to facilitate navigation in the code of this branch.) This formalization is outlined in the paper _Formalization of derived categories in Lean/mathlib_ https://hal.science/hal-04546712 The homology of `ShortComplex C` (diagrams of two composable morphisms whose composition is zero) is developed in `Algebra.Homology.ShortComplex`. The files in that folder have been added one by one in separate PRs, and then, the current definition of `homology` has been replaced by this new definition in a refactor PR.
Homology refactor: * #4203 * #4204 * #4388 * #4609 * #4645 * #4787 * #4853 * #5250 * #5674 * #6008 * #6039 * #6089 * #6227 * #6230 * #6231 * #6245 * #6267 * #6279 * #6324 * #6443 * #6586 * #6994 * #7042 * #7047 * #7052 * #7192 * #7193 * #7194 * #7195 * #7197 * #7256 * #7262 * #7280 * #7623 * #7624 * #7806 * #7816 * #7817 * #7821 * #7954 * #7966 * #7993 * #7995 * #7996 * #7997 * #8058 * #8060 * #8069 * #8079 * #8081 * #8084 * #8091 * #8113 * #8114 * #8152 * #8159 * #8174 * #8200 * #8206 * #8208 * #8472 * #8468 * #8475 * #8490 * #8491 * #8507 * #8512 * #8593 * #8595 * #8706 * #8765 * #8766 * #8845 * #9022 * #12649 * #12638
Homological complexes: * #9333 * #9335 * #9331
Localization of categories: * #6233 * #6235 * #6236 * #6867 * #6869 * #6887 * #6882 * #8041 * #8055 * #8069 * #8516 * #8864 * #8865 * #9702 * #9692 * #10606 * #10607 * #11721 * #11728 * #11737 * #12728
Shifts on categories: * #4429 * #6652 * #6653 * #6655 * #7268 * #7270 * #9001 * #11764
Triangulated categories: * #6377 * #6688 * #6815 * #7053 * #7324 * #7327 * #7336 * #7626 * #7641 * #9049 * #9073 * #10527 * #11738 * #11740 * #11759 * #11786 * #11789 * #11805 * #12619
Construction of the derived category: * #6626 * #6701 * #6720 * #6894 * #7048 * #7049 * #7050 * #7201 * #7656 * #8937 * #8966 * #8969 * #8970 * #9054 * #9447 * #8951 * #9483 * #9508 * #9509 * #9592 * #9614 * #9615 * #9032 * #9370 * #9550 * #9686 * #9660 * #11760 * #11782 * #11806
Derived functors: * #10195 * #10270 * #10301 * #10384 * #10413 * #12168 * #12627 * #12631 * #12633 * #12785 * #12788
Refactor of Ext-groups: * #12607
- [ ] depends on: #24309 - [ ] depends on: #24275 - [ ] depends on: #24191 - [ ] depends on: #23797 - [ ] depends on: #22586 - [ ] depends on: #22556 - [ ] depends on: #22547 - [ ] depends on: #22539 - [ ] depends on: #22508 - [ ] depends on: #22450 - [ ] depends on: #23915 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/)
large-import t-topology t-category-theory merge-conflict blocked-by-other-PR WIP 41980/508 Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Free.lean,Mathlib/Algebra/Category/ModuleCat/LeftResolutions.lean,Mathlib/Algebra/Homology/Additive.lean,Mathlib/Algebra/Homology/BicomplexColumns.lean,Mathlib/Algebra/Homology/BicomplexRows.lean,Mathlib/Algebra/Homology/Bifunctor.lean,Mathlib/Algebra/Homology/BifunctorColimits.lean,Mathlib/Algebra/Homology/BifunctorCommShift.lean,Mathlib/Algebra/Homology/BifunctorFlip.lean,Mathlib/Algebra/Homology/BifunctorHomotopy.lean,Mathlib/Algebra/Homology/BifunctorMappingCone.lean,Mathlib/Algebra/Homology/BifunctorShift.lean,Mathlib/Algebra/Homology/BifunctorSingle.lean,Mathlib/Algebra/Homology/BifunctorTriangulated.lean,Mathlib/Algebra/Homology/CategoryWithHomology.lean,Mathlib/Algebra/Homology/CochainComplexMinus.lean,Mathlib/Algebra/Homology/ComplexShape.lean,Mathlib/Algebra/Homology/ComplexShapeSigns.lean,Mathlib/Algebra/Homology/ConnectShortExact.lean,Mathlib/Algebra/Homology/DerivedCategory/Basic.lean,Mathlib/Algebra/Homology/DerivedCategory/DerivabilityStructureInjectives.lean,Mathlib/Algebra/Homology/DerivedCategory/Ext/Linear.lean,Mathlib/Algebra/Homology/DerivedCategory/Fractions.lean,Mathlib/Algebra/Homology/DerivedCategory/FullyFaithful.lean,Mathlib/Algebra/Homology/DerivedCategory/HomologySequence.lean,Mathlib/Algebra/Homology/DerivedCategory/Linear.lean,Mathlib/Algebra/Homology/DerivedCategory/Minus.lean,Mathlib/Algebra/Homology/DerivedCategory/Monoidal.lean,Mathlib/Algebra/Homology/DerivedCategory/Plus.lean,Mathlib/Algebra/Homology/DerivedCategory/RightDerivedFunctorPlus.lean,Mathlib/Algebra/Homology/DerivedCategory/SingleTriangle.lean,Mathlib/Algebra/Homology/DerivedCategory/SpectralObject.lean,Mathlib/Algebra/Homology/DerivedCategory/TStructure.lean,Mathlib/Algebra/Homology/Double.lean,Mathlib/Algebra/Homology/DoubleHomology.lean,Mathlib/Algebra/Homology/Embedding/Boundary.lean,Mathlib/Algebra/Homology/Embedding/CochainComplex.lean,Mathlib/Algebra/Homology/Embedding/CochainComplexTrunc.lean,Mathlib/Algebra/Homology/Embedding/ComplementaryTrunc.lean,Mathlib/Algebra/Homology/Embedding/ExtendMap.lean,Mathlib/Algebra/Homology/Embedding/HomEquiv.lean,Mathlib/Algebra/Homology/Embedding/StupidFiltration.lean,Mathlib/Algebra/Homology/Embedding/StupidTrunc.lean,Mathlib/Algebra/Homology/Embedding/TruncGE.lean,Mathlib/Algebra/Homology/Embedding/TruncLE.lean,Mathlib/Algebra/Homology/Embedding/TruncLEHomology.lean,Mathlib/Algebra/Homology/ExactSequence.lean,Mathlib/Algebra/Homology/ExactSequenceFour.lean,Mathlib/Algebra/Homology/Factorizations/Basic.lean,Mathlib/Algebra/Homology/Factorizations/CM5a.lean,Mathlib/Algebra/Homology/Factorizations/CM5b.lean,Mathlib/Algebra/Homology/HomologicalBicomplex.lean,Mathlib/Algebra/Homology/HomologicalComplex.lean,Mathlib/Algebra/Homology/HomologicalComplexFunctorEquiv.lean,Mathlib/Algebra/Homology/HomologicalComplexLimits.lean,Mathlib/Algebra/Homology/HomologicalComplexLimitsEventuallyConstant.lean,Mathlib/Algebra/Homology/Homology.lean,Mathlib/Algebra/Homology/HomologySequence.lean,Mathlib/Algebra/Homology/HomologySequenceLemmas.lean,Mathlib/Algebra/Homology/Homotopy.lean,Mathlib/Algebra/Homology/HomotopyCategory.lean,Mathlib/Algebra/Homology/HomotopyCategory/Cylinder.lean,Mathlib/Algebra/Homology/HomotopyCategory/DegreewiseSplit.lean,Mathlib/Algebra/Homology/HomotopyCategory/Devissage.lean,Mathlib/Algebra/Homology/HomotopyCategory/HomComplex.lean,Mathlib/Algebra/Homology/HomotopyCategory/HomComplexShift.lean,Mathlib/Algebra/Homology/HomotopyCategory/KInjective.lean,Mathlib/Algebra/Homology/HomotopyCategory/MappingCone.lean,Mathlib/Algebra/Homology/HomotopyCategory/Minus.lean,Mathlib/Algebra/Homology/HomotopyCategory/Monoidal.lean,Mathlib/Algebra/Homology/HomotopyCategory/MonoidalTriangulated.lean,Mathlib/Algebra/Homology/HomotopyCategory/Plus.lean,Mathlib/Algebra/Homology/HomotopyCategory/PreservesQuasiIso.lean,Mathlib/Algebra/Homology/HomotopyCategory/Pretriangulated.lean,Mathlib/Algebra/Homology/HomotopyCategory/Shift.lean,Mathlib/Algebra/Homology/HomotopyCategory/ShiftSequence.lean,Mathlib/Algebra/Homology/HomotopyCategory/ShortExact.lean,Mathlib/Algebra/Homology/HomotopyCategory/SingleFunctors.lean,Mathlib/Algebra/Homology/HomotopyCategory/SpectralObject.lean,Mathlib/Algebra/Homology/HomotopyFiber.lean,Mathlib/Algebra/Homology/LeftResolutions/Basic.lean,Mathlib/Algebra/Homology/LeftResolutions/CochainComplex.lean,Mathlib/Algebra/Homology/LeftResolutions/CochainComplexMinus.lean,Mathlib/Algebra/Homology/LeftResolutions/Reduced.lean,Mathlib/Algebra/Homology/LeftResolutions/Transport.lean,Mathlib/Algebra/Homology/Localization.lean,Mathlib/Algebra/Homology/Monoidal.lean,Mathlib/Algebra/Homology/ObjectProperty.lean,Mathlib/Algebra/Homology/PreservesQuasiIso.lean,Mathlib/Algebra/Homology/QuasiIso.lean,Mathlib/Algebra/Homology/Refinements.lean,Mathlib/Algebra/Homology/ShortComplex/Abelian.lean,Mathlib/Algebra/Homology/ShortComplex/Basic.lean,Mathlib/Algebra/Homology/ShortComplex/Exact.lean,Mathlib/Algebra/Homology/ShortComplex/FiveLemma.lean,Mathlib/Algebra/Homology/ShortComplex/FourLemma.lean,Mathlib/Algebra/Homology/ShortComplex/HomologicalComplex.lean,Mathlib/Algebra/Homology/ShortComplex/Images.lean,Mathlib/Algebra/Homology/ShortComplex/Preadditive.lean 299 n/a ['digama0', 'github-actions', 'jcommelin', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
25-85079
25 days ago
unknown
unknown
13685 niklasmohrin
author:niklasmohrin
feat(Combinatorics): add definitions for network flows Although we might not have any super-interesting results ready for mathlib yet, I feel that the definitions from this commit are already mature enough to include. These definitions are ported from last semester's work we did at https://github.com/niklasmohrin/lean-seminar-2023 and I have put some time in to refactor our code to `Int` and now to any parameter `R`. In the linked repository, there is some more stuff that I can send in. One obstacle without integer values is that it is not clear why a maximum flow would exist. I think the best way to tackle this would be to prove max-flow-min-cut theorem and implement the Ford-Fulkerson algorithm. It has been pointed out on Zulip that there is an [Isabelle formalization of the Edmonds Karp Algorithm](https://www.isa-afp.org/entries/EdmondsKarp_Maxflow.html). I feel that the definitions are pretty solid and it makes sense to include them, even if just for unifying definitions across downstream projects. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-combinatorics merge-conflict awaiting-author 244/0 Mathlib.lean,Mathlib/Combinatorics/Flow/Basic.lean,docs/references.bib 3 57 ['Shreyas4991', 'YaelDillies', 'b-mehta', 'github-actions', 'leanprover-community-bot-assistant', 'madvorak', 'niklasmohrin'] nobody
25-70063
25 days ago
25-70065
25 days ago
86-21072
86 days
24208 ADedecker
author:ADedecker
chore: semilinearize LinearAlgebra.TensorProduct.Basic This was painful, and it's not without consequences, but this is necessary in order to talk about tensor products of Hilbert spaces. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict WIP
label:t-algebra$
191/138 Mathlib/Algebra/Category/ModuleCat/ChangeOfRings.lean,Mathlib/Algebra/Category/ModuleCat/Monoidal/Closed.lean,Mathlib/Algebra/Lie/TensorProduct.lean,Mathlib/Algebra/Module/Equiv/Defs.lean,Mathlib/LinearAlgebra/BilinearForm/TensorProduct.lean,Mathlib/LinearAlgebra/BilinearMap.lean,Mathlib/LinearAlgebra/Dual/Lemmas.lean,Mathlib/LinearAlgebra/TensorPower/Basic.lean,Mathlib/LinearAlgebra/TensorProduct/Associator.lean,Mathlib/LinearAlgebra/TensorProduct/Basic.lean,Mathlib/LinearAlgebra/TensorProduct/Tower.lean,Mathlib/RingTheory/Coalgebra/Hom.lean 12 2 ['github-actions', 'leanprover-community-bot-assistant'] nobody
25-56110
25 days ago
25-56111
25 days ago
0-25
25 seconds
15115 kkytola
author:kkytola
feat: Generalize assumptions in liminf and limsup results in ENNReals In a [review comment](https://github.com/leanprover-community/mathlib4/pull/13938#discussion_r1649744441) it was pointed out that results about liminf and limsup in ENNReal hold under milder assumptions. This PR does the generalization. --- This PR is split off from #13938, where the review comment was made. The changes needed for the suggested generalization were of different kind than the simple PR's content, justifying a separate PR. - [x] depends on: #13938 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order t-topology merge-conflict awaiting-author help-wanted 215/27 Mathlib/MeasureTheory/Measure/Portmanteau.lean,Mathlib/Order/LiminfLimsup.lean,Mathlib/Topology/Instances/ENNReal.lean 3 8 ['Ruben-VandeVelde', 'github-actions', 'grunweg', 'j-loreaux', 'kkytola', 'leanprover-community-mathlib4-bot'] nobody
25-25819
25 days ago
50-10123
1 month ago
21-25493
21 days
21603 imbrem
author:imbrem
feat(CategoryTheory/ChosenFiniteProducts): add basic ChosenFiniteCoproducts class Added basic `ChosenFiniteCoproducts` class, and started porting some of the lemmas about `ChosenFiniteProducts` suitably translated --- This, combined with #20182 modified to use chosen finite coproducts and premonoidal categories (#21488), should be enough for me to formalize strong Elgot categories, and hence a lot of categorical iteration theory for my PhD thesis. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-category-theory merge-conflict awaiting-author 261/2 Mathlib/CategoryTheory/ChosenFiniteProducts.lean 1 17 ['TwoFX', 'YaelDillies', 'github-actions', 'grunweg', 'imbrem', 'joelriou', 'leanprover-community-bot-assistant'] TwoFX and joelriou
assignee:TwoFX assignee:joelriou
25-2480
25 days ago
25-2662
25 days ago
89-21170
89 days
22639 b-reinke
author:b-reinke
feat(Mathlib/GroupTheory/FreeGroup): theory of (cyclically) reduced words Upstreamed from the [EquationalTheories](https://github.com/teorth/equational_theories) project. This PR defines in the new file `Mathlib/GroupTheory/FreeGroup/ReducedWords.lean` some extra lemmas for free groups, in particular about (cyclically) reduced words. ## Main declarations * `FreeGroup.Red.reduced`: the predicate for reduced words * `FreeGroup.Red.cyclicallyReduced`: the predicate for cyclically reduced words ## Main statements * `FreeGroup.infinite_order`: nontrivial elements of a free group have infinite order * `FreeGroup.zpow_left_injective`: taking n-th powers is an injective function on the free group Co-authored-by: Amir Livne Bar-on - [ ] depends on: #23366 - [ ] depends on: #23367 - [ ] depends on: #23368 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra merge-conflict blocked-by-other-PR
label:t-algebra$
429/0 Mathlib.lean,Mathlib/GroupTheory/FreeGroup/Basic.lean,Mathlib/GroupTheory/FreeGroup/Reduce.lean,Mathlib/GroupTheory/FreeGroup/ReducedWords.lean 4 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
24-45371
24 days ago
24-45374
24 days ago
20-75471
20 days
17129 joneugster
author:joneugster
feat(Tactic/Linter): add unicode linter for unicode variant-selectors Unicode characters can be followed by one of the two "variant-selectors" `\FE0E` (text) or `\FE0F` (emoji). These appear to the user as a single unicode character and they might copy them by accident. For example `✅️` (`\u2705\uFE0F`), `✅` (`\u2705`) and `✅︎` (`\u2705\uFE0E`) are three variants of the "same" unicode character. The one without variant-selector might display as either emoji or not, depending on the user's device and font. Add unicode linter ensuring variant-selector only appear on specified characters and also ensuring these characters always have the correct variant selector to avoid confusions. Everything flagged by this linter can be fixed fully automatically with `lake exe lint-style --fix` or by commenting `bot fix style` on the PR. --- - tracking PR: #16215 ## Zulip discussions: - https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/Whitelist.20for.20Unicode.3F - https://leanprover.zulipchat.com/#narrow/stream/113488-general/topic/Lean.20specific.20font ## Related PRs: - leanprover/lean4#5015 added some emoji-variant selectors to Emojis used in `Lean` itself. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-linter merge-conflict delegated awaiting-author 245/14 Mathlib.lean,Mathlib/GroupTheory/GroupExtension/Defs.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter/TextBased.lean,Mathlib/Tactic/Linter/UnicodeLinter.lean,Mathlib/Tactic/Widget/Calc.lean,Mathlib/Tactic/Widget/CongrM.lean,Mathlib/Tactic/Widget/Conv.lean,Mathlib/Tactic/Widget/GCongr.lean,Mathlib/Topology/ContinuousMap/Weierstrass.lean,MathlibTest/LintStyleTextBased.lean 11 25 ['YaelDillies', 'adomani', 'github-actions', 'grunweg', 'joneugster', 'kim-em', 'leanprover-community-bot-assistant'] nobody
24-14325
24 days ago
24-14327
24 days ago
82-54712
82 days
17131 joneugster
author:joneugster
feat(Tactic/Linter): add unicode linter for unwanted characters Add unicode linter flagging bad unicode characters. In this first form, the linter only flags `\u00A0` (non-breaking space) and replaces it with a normal space. Non-breaking space has been chosen because they keep reappearing in mathlib and it seems to be uncontroversial to lint for these. The whitelist/blacklist could then be refined in future PRs. Everything flagged by this linter can be fixed fully automatically with `lake exe lint-style --fix` or by commenting `bot fix style` on the PR. --- - tracking PR: #16215 ## Zulip discussions: - https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/Whitelist.20for.20Unicode.3F - https://leanprover.zulipchat.com/#narrow/stream/113488-general/topic/Lean.20specific.20font [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-linter merge-conflict awaiting-author 112/8 Mathlib.lean,Mathlib/Algebra/Lie/Semisimple/Lemmas.lean,Mathlib/Analysis/Analytic/IsolatedZeros.lean,Mathlib/CategoryTheory/Category/ReflQuiv.lean,Mathlib/LinearAlgebra/Vandermonde.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter/TextBased.lean,Mathlib/Tactic/Linter/UnicodeLinter.lean 8 6 ['github-actions', 'grunweg', 'leanprover-community-bot-assistant'] adomani and grunweg
assignee:grunweg assignee:adomani
24-14324
24 days ago
24-14326
24 days ago
52-18594
52 days
8495 jjaassoonn
author:jjaassoonn
feat : Tensor-Hom adjunction in the category of modules # Tensor-Hom adjunction Let $R$ be a commutative ring and $S$ any ring. Let $X$ be an $(S,R)$-bimoule. Then the tensor functor $(X \otimes_R \cdot)$ is a functor from left $R$-modules to left $S$-modules; and the hom-functor $Hom_S(X, \cdot)$ is a functor from left $S$-modules to left $R$-modules. For another left $S$-module $Y$, the left $R$-module structure of $Hom_S(X, Y)$ is given by $s \cdot f := x \mapsto f(s \cdot x)$. These two functors are adjoint.. In particular we have that ```math {\rm Hom}_{S}(X\otimes_R Y, Z) \cong {\rm Hom}_R (Y, {\rm Hom}_S (X, Z)) ``` ## Implementation notes 1. Why not use the `Mathlib/LinearAlgebra/TensorProduct/Tower.lean` In our setting `X` is an `(R, S)` bimodule and `Y` an `R`-module and `Z` an `S`-module so to use the `Tower` file, we need `S` to be an `R`-algebra which is a luxury we do not have. But note that in `Tower` file, `curry` and `uncurry` are both tri-linear maps. So `Tower` file allows interplay of 3 rings which is not allowed in this file. 2. We require `R` to be commutative but we never used anything commutative. This is because of tensor product requires commutativity, but thanks to @alreadydone, this assumption could be removed soon. I think this PR should wait for Junyan's attempt on removing commutativity, so it is marked as draft and wip for now --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict awaiting-author WIP
label:t-algebra$
214/0 Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/TensorHomAdjunction.lean 2 88 ['alreadydone', 'bustercopley', 'eric-wieser', 'github-actions', 'jjaassoonn', 'kbuzzard', 'kim-em', 'leanprover-community-bot-assistant'] eric-wieser
assignee:eric-wieser
23-20355
23 days ago
23-20356
23 days ago
0-0
0 seconds
24590 smmercuri
author:smmercuri
chore: make `Valuation.Completion` a `def` and refactor more of `AdicValuation.lean` The main purpose of this PR is to resolve timeout issues encountered in FLT following the refactor of `HeightOneSpectrum.adicCompletion` to use the `WithVal` type synonym. The proposed fix in this PR is to replace `abbrev` with `def` in `Valuation.Completion`. Tested in FLT and this removes the timeout issue. Also refactor as much API as possible from `HeightOneSpectrum.adicCompletion` to `Valuation.Completion`. See #22488 for a previous attempt at fixing the problem. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) FLT merge-conflict 162/81 Mathlib/NumberTheory/NumberField/FinitePlaces.lean,Mathlib/RingTheory/DedekindDomain/AdicValuation.lean,Mathlib/RingTheory/DedekindDomain/FiniteAdeleRing.lean,Mathlib/RingTheory/LaurentSeries.lean,Mathlib/Topology/Algebra/Valued/WithVal.lean 5 5 ['github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'smmercuri'] nobody
22-78761
22 days ago
22-78763
22 days ago
13-35725
13 days
19284 adomani
author:adomani
test: commit a change only to the "master" CI build action This PR should fail CI, since the main CI build file is incompatible with the autogenerated ones. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) CI merge-conflict awaiting-author 3/3 .github/build.in.yml,.github/workflows/actionlint.yml 2 12 ['adomani', 'bryangingechen', 'github-actions', 'jcommelin', 'leanprover-community-bot-assistant'] bryangingechen
assignee:bryangingechen
21-51759
21 days ago
21-51760
21 days ago
0-0
0 seconds
15651 TpmKranz
author:TpmKranz
feat(Computability/NFA): operations for Thompson's construction Lays the groundwork for a proof of equivalence of RE and NFA, w.r.t. described language. Actual connection to REs comes later, after the groundwork for the opposite direction has been laid. Third chunk of #12648 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-zulip t-computability new-contributor merge-conflict awaiting-author 307/5 Mathlib/Computability/NFA.lean 1 15 ['TpmKranz', 'YaelDillies', 'dupuisf', 'github-actions', 'leanprover-community-bot-assistant', 'meithecatte'] nobody
21-14071
21 days ago
21-14072
21 days ago
45-84611
45 days
22361 rudynicolop
author:rudynicolop
feat(Computability/NFA): nfa closure properties Add the closure properties union, intersection and reversal for NFA. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-zulip t-computability new-contributor merge-conflict awaiting-author 218/2 Mathlib/Computability/Language.lean,Mathlib/Computability/NFA.lean 2 90 ['EtienneC30', 'b-mehta', 'github-actions', 'leanprover-community-bot-assistant', 'meithecatte', 'rudynicolop'] EtienneC30
assignee:EtienneC30
21-13145
21 days ago
21-13147
21 days ago
39-67601
39 days
21255 chrisflav
author:chrisflav
feat(RingTheory/Smooth): smooth is equivalent to locally standard smooth This is only a container to not lose the branch name. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict
label:t-algebra$
1740/11 Mathlib.lean,Mathlib/RingTheory/Kaehler/Localization.lean,Mathlib/RingTheory/Presentation.lean,Mathlib/RingTheory/Smooth/FreeKaehler.lean,Mathlib/RingTheory/Smooth/StandardSmoothCotangent.lean,Mathlib/RingTheory/Smooth/StandardSmoothSmooth.lean 6 2 ['github-actions', 'leanprover-community-bot-assistant'] nobody
20-42508
20 days ago
20-42510
20 days ago
0-0
0 seconds
23281 mattrobball
author:mattrobball
test merge-conflict 12/10 Mathlib/AlgebraicGeometry/Cover/Open.lean,Mathlib/Analysis/Normed/Unbundled/SeminormFromConst.lean,Mathlib/FieldTheory/IntermediateField/Adjoin/Basic.lean,Mathlib/Order/Part.lean,Mathlib/RingTheory/Extension.lean,Mathlib/RingTheory/Kaehler/CotangentComplex.lean,Mathlib/Topology/Category/TopCat/Limits/Basic.lean 7 5 ['github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'mattrobball'] nobody
20-39889
20 days ago
20-39891
20 days ago
0-0
0 seconds
24245 JovanGerb
author:JovanGerb
feat(Geometry/Euclidean/SignedDist): `signedDist` between two points This PR defines `signedDist`, the signed distance between two points. It redefines `signedInfDist` so that it uses `signedDist`. The motivation is to use this in IMO2020Q6. Additionally this definition will be useful for properly reasoning about the power of a point [#mathlib4 > Signed distance between points](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Signed.20distance.20between.20points) some comments: * should `signedDistLinear` be `private`? * should `signedDist` and `signedInfDist` be made continuous bunled maps in this PR? * I'm not too happy about the hypothesis in `signedDist_congr (h : ∃ r > (0 : ℝ), r • v = w)`. This relationship between `v` and `w` is a symmetric one that should have some API around it, similar to `SameRay`. It could also be spelled as `(ℝ≥0 ∙ v) = ℝ≥0 ∙ w` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-euclidean-geometry merge-conflict 206/23 Mathlib/Analysis/InnerProductSpace/Basic.lean,Mathlib/Geometry/Euclidean/SignedDist.lean,Mathlib/Topology/MetricSpace/Pseudo/Defs.lean 3 2 ['github-actions', 'leanprover-community-bot-assistant'] nobody
18-84326
18 days ago
18-84328
18 days ago
30-61949
30 days
18486 vasnesterov
author:vasnesterov
feat(Tactic): tactic for computing asymptotics of real functions It's an auxiliary PR which implements the entire `compute_asymptotics` tactic. I will split it into multiple small PRs. --- In this PR I implement the `compute_asymptotics` tactic. Its purpose is to compute asymptotics of functions from `ℝ` to `ℝ`. So far it is able to compute the limit of any function constructed using arithmetic operations (`+`, `-`, `*`, `/`, inversion) and powers with constant real exponent. ```lean example : let f := fun (x : ℝ) ↦ (4 * x)/(3 + 2 * x); Tendsto f atTop (nhds 2) := by simp only compute_asymptotics example : let f := fun (x : ℝ) ↦ x^(1/2 : ℝ) / (x^(1/3 : ℝ) + x^(-1/3 : ℝ) + 18); Tendsto f atTop atTop := by simp only compute_asymptotics ``` It also supports non-numerical constants: ```lean example (a : ℝ) (h : 0 < a) : let f := fun (x : ℝ) ↦ a * x; Tendsto f atTop atTop := by simp only compute_asymptotics example : let f := fun (x : ℝ) ↦ Real.pi * x; Tendsto f atTop atTop := by simp only have : 0 < Real.pi := Real.pi_pos compute_asymptotics ``` (for more examples see `compute_asymptotics.lean` in tests) ### Isn't it undecidable? In general, finding the limit of a given function is undecidable problem, due to undecidability of the problem of comparing real numbers. So far I use `linarith` tactic for this under the hood. When it's unable to prove neither of `x < y`, `y < x`, `x = y`, the tactic fails. ### TODO * Prove the goals of the form `f =o[l] g` and similarly for other O-notations. * Add `sin`, `cos`, `exp`, and `log` support. ### References I am basically implementing [this article](https://www21.in.tum.de/~eberlm/pdfs/real_asymp.pdf) about computing asymptotics in Isabelle by Manuel Eberl. - [ ] depends on: #22531 - [ ] depends on: #23790 - [x] depends on: #23748 - [ ] depends on: #23749 - [ ] depends on: #22538 - [ ] depends on: #23831 - [ ] depends on: #22531 - [x] depends on: #20071 - [ ] depends on: #20160 - [ ] depends on: #20241 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta merge-conflict blocked-by-other-PR WIP 11886/331 Mathlib.lean,Mathlib/Analysis/Calculus/FDeriv/Analytic.lean,Mathlib/Analysis/Calculus/FormalMultilinearSeries.lean,Mathlib/Data/Seq/Parallel.lean,Mathlib/Data/Seq/Seq.lean,Mathlib/Data/Set/Pointwise/Interval.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Tendsto/Lemmas.lean,Mathlib/Tactic/Tendsto/Main.lean,Mathlib/Tactic/Tendsto/Meta/CompareReal.lean,Mathlib/Tactic/Tendsto/Meta/ConstSimp.lean,Mathlib/Tactic/Tendsto/Meta/Defs.lean,Mathlib/Tactic/Tendsto/Meta/ElimDestruct.lean,Mathlib/Tactic/Tendsto/Meta/LeadingTerm.lean,Mathlib/Tactic/Tendsto/Meta/MS.lean,Mathlib/Tactic/Tendsto/Meta/Main.lean,Mathlib/Tactic/Tendsto/Meta/Trimming.lean,Mathlib/Tactic/Tendsto/Multiseries.lean,Mathlib/Tactic/Tendsto/Multiseries/Basic.lean,Mathlib/Tactic/Tendsto/Multiseries/Basis.lean,Mathlib/Tactic/Tendsto/Multiseries/Defs.lean,Mathlib/Tactic/Tendsto/Multiseries/LeadingTerm.lean,Mathlib/Tactic/Tendsto/Multiseries/Operations.lean,Mathlib/Tactic/Tendsto/Multiseries/Operations/Add.lean,Mathlib/Tactic/Tendsto/Multiseries/Operations/Basic.lean,Mathlib/Tactic/Tendsto/Multiseries/Operations/ForPow.lean,Mathlib/Tactic/Tendsto/Multiseries/Operations/Inv.lean,Mathlib/Tactic/Tendsto/Multiseries/Operations/Merge.lean,Mathlib/Tactic/Tendsto/Multiseries/Operations/Mul.lean,Mathlib/Tactic/Tendsto/Multiseries/Operations/Pow.lean,Mathlib/Tactic/Tendsto/Multiseries/Operations/Powser.lean,Mathlib/Tactic/Tendsto/Multiseries/Term.lean,Mathlib/Tactic/Tendsto/Multiseries/Trimming.lean,Mathlib/Topology/Algebra/Order/Field.lean,MathlibTest/compute_asymptotics.lean,MathlibTest/kek.lean 36 55 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
18-12138
18 days ago
32-22636
1 month ago
0-0
0 seconds
15254 yuma-mizuno
author:yuma-mizuno
feat(CategoryTheory/Monoidal): replace `Mon_` lemmas with `Mon_Class` lemmas We redefine algebras internal to monoidal categories, which were defined by full-bundled structures, in terms of semi-bundled type classes. The original full-bundled structure `X` is renamed to `X_Cat`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory merge-conflict WIP 3982/96 Mathlib.lean,Mathlib/CategoryTheory/Monoidal/Bimod_Class.lean,Mathlib/CategoryTheory/Monoidal/Bimon_.lean,Mathlib/CategoryTheory/Monoidal/Bimon_Class copy.lean,Mathlib/CategoryTheory/Monoidal/Bimon_Class.lean,Mathlib/CategoryTheory/Monoidal/Braided/Opposite.lean,Mathlib/CategoryTheory/Monoidal/CommMon_Class.lean,Mathlib/CategoryTheory/Monoidal/Comon_.lean,Mathlib/CategoryTheory/Monoidal/Comon_Class.lean,Mathlib/CategoryTheory/Monoidal/Internal/ModuleClass.lean,Mathlib/CategoryTheory/Monoidal/Mod_Class.lean,Mathlib/CategoryTheory/Monoidal/Mon_.lean,Mathlib/CategoryTheory/Monoidal/Mon_Class.lean,Mathlib/CategoryTheory/Monoidal/mwe.lean 14 n/a ['YaelDillies', 'github-actions', 'leanprover-community-bot-assistant', 'yuma-mizuno'] nobody
17-77330
17 days ago
unknown
unknown
25006 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 This is a preparatory PR for [#24849](https://github.com/leanprover-community/mathlib4/pull/24849) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict awaiting-author
label:t-algebra$
214/0 Mathlib/Algebra/Lie/Weights/RootSystem.lean 1 3 ['github-actions', 'leanprover-community-bot-assistant', 'ocfnash'] nobody
17-38419
17 days ago
20-83831
20 days ago
1-1321
1 day
21760 101damnations
author:101damnations
feat(RepresentationTheory/GroupCohomology/LongExactSequence): specialise LES API to group cohomology Given a commutative ring `k` and a group `G`, this PR shows that a short exact sequence of `k`-linear `G`-representations `0 ⟶ X₁ ⟶ X₂ ⟶ X₃ ⟶ 0` induces a short exact sequence of complexes of inhomogeneous cochains `0 ⟶ C(X₁) ⟶ C(X₂) ⟶ C(X₃) ⟶ 0`, where `Hⁿ(C(Xᵢ))` is the `n`th group cohomology of `Xᵢ`. This allows us to specialize API about long exact sequences to group cohomology. --- - [x] depends on: #21652 - [x] depends on: #21739 - [x] depends on: #21756 - [x] depends on: #21758 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-category-theory merge-conflict awaiting-author WIP
label:t-algebra$
1247/83 Mathlib.lean,Mathlib/Algebra/Homology/ConcreteCategory.lean,Mathlib/Algebra/Homology/HomologySequence.lean,Mathlib/Algebra/Homology/ShortComplex/ModuleCat.lean,Mathlib/Algebra/Homology/ShortComplex/SnakeLemma.lean,Mathlib/LinearAlgebra/Pi.lean,Mathlib/RepresentationTheory/GroupCohomology/Functoriality.lean,Mathlib/RepresentationTheory/GroupCohomology/LongExactSequence.lean,Mathlib/RepresentationTheory/GroupCohomology/LowDegree.lean,Mathlib/RepresentationTheory/GroupCohomology/ToMove.lean 10 6 ['github-actions', 'joelriou', 'kbuzzard', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
17-30220
17 days ago
17-30221
17 days ago
15-42431
15 days
21765 101damnations
author:101damnations
feat(RepresentationTheory/GroupCohomology/LongExactSequence): specialise LES API to low degree group cohomology Given a commutative ring `k` and a group `G`, this file shows that a short exact sequence of `k`-linear `G`-representations `0 ⟶ X₁ ⟶ X₂ ⟶ X₃ ⟶ 0` induces a short exact sequence of complexes of inhomogeneous cochains `0 ⟶ C(X₁) ⟶ C(X₂) ⟶ C(X₃) ⟶ 0`, where `Hⁿ(C(Xᵢ))` is the `n`th group cohomology of `Xᵢ`. This allows us to specialize API about long exact sequences to group cohomology; in this PR we focus on degrees `n = 0, 1, 2`. --- - [x] depends on: #21652 - [x] depends on: #21739 - [x] depends on: #21756 - [x] depends on: #21758 - [ ] depends on: #21760 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict blocked-by-other-PR
label:t-algebra$
554/91 Mathlib.lean,Mathlib/Algebra/Homology/ConcreteCategory.lean,Mathlib/Algebra/Homology/HomologySequence.lean,Mathlib/Algebra/Homology/ShortComplex/ModuleCat.lean,Mathlib/Algebra/Homology/ShortComplex/SnakeLemma.lean,Mathlib/LinearAlgebra/Pi.lean,Mathlib/RepresentationTheory/GroupCohomology/Basic.lean,Mathlib/RepresentationTheory/GroupCohomology/Functoriality.lean,Mathlib/RepresentationTheory/GroupCohomology/LongExactSequence.lean,Mathlib/RepresentationTheory/GroupCohomology/LowDegree.lean 10 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
17-30218
17 days ago
17-30220
17 days ago
0-309
5 minutes
20733 winstonyin
author:winstonyin
feat: solution to ODE is Lipschitz with respect to the initial condition I formalise a corollary to the Picard-Lindelöf theorem: the local solution to an ODE is Lipschitz continuous with respect to the initial condition. This in particular means that the local flow to the associated vector field is continuous. - [ ] depends on: #20704 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-dynamics t-analysis merge-conflict blocked-by-other-PR 688/360 Mathlib/Algebra/Order/Group/Abs.lean,Mathlib/Analysis/Normed/Group/Basic.lean,Mathlib/Analysis/ODE/PicardLindelof.lean,Mathlib/Geometry/Manifold/IntegralCurve/ExistUnique.lean,docs/1000.yaml,docs/undergrad.yaml 6 5 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
16-65045
16 days ago
16-65046
16 days ago
0-1005
16 minutes
21286 winstonyin
author:winstonyin
feat: solutions to $C^n$ vector fields are $C^n$ in time I prove that solutions to $C^n$ vector fields are also $C^n$ in time, where $n ≤ \infty$. - [ ] depends on: #20733 [technically only depends on #20704 but I'm writing these as incremental PRs] --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-dynamics t-analysis merge-conflict blocked-by-other-PR 795/360 Mathlib/Algebra/Order/Group/Abs.lean,Mathlib/Analysis/Normed/Group/Basic.lean,Mathlib/Analysis/ODE/PicardLindelof.lean,Mathlib/Geometry/Manifold/IntegralCurve/ExistUnique.lean,docs/1000.yaml,docs/undergrad.yaml 6 6 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
16-65044
16 days ago
16-65046
16 days ago
0-298
4 minutes
21777 winstonyin
author:winstonyin
feat: existence of local flows on manifolds Transfer the existence theorem of local flows on vector spaces to manifolds. The precise statement is: > If a vector field `v` on a manifold `M` is continuously differentiable at an interior point `x₀`, then for a given `t₀` there exists a neighbourhood `u` of `x₀`, a positive `ε`, and `γ : M → ℝ → M` such that `γ x` is an integral curve of `v` on `(t₀ - ε, t₀ + ε)` for all `x ∈ u`. This is powerful because all curves `γ x` (each with initial condition `x ∈ u`) share the same existence time interval `(t₀ - ε, t₀ + ε)`, rather than each curve having its own `ε`. This will allow us to show that $C^1$ vector fields on compact manifolds always have global integral curves / global flows. Any suggestions to shorten the proof or split out useful lemmas are welcome! - [ ] depends on: #20733 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-differential-geometry merge-conflict blocked-by-other-PR WIP 2223/408 Mathlib/Algebra/Order/Group/Abs.lean,Mathlib/Analysis/Normed/Group/Basic.lean,Mathlib/Analysis/ODE/PicardLindelof new.lean,Mathlib/Analysis/ODE/PicardLindelof old.lean,Mathlib/Analysis/ODE/PicardLindelof.lean,Mathlib/Geometry/Manifold/IntegralCurve/ExistUnique.lean,Mathlib/Order/Filter/Prod.lean,docs/1000.yaml,docs/undergrad.yaml 9 5 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
16-64920
16 days ago
16-64922
16 days ago
0-0
0 seconds
22254 winstonyin
author:winstonyin
feat: $C^1$ vector fields on compact manifolds define global flows Any $C^1$ vector field on a compact boundaryless manifold `M` defines a unique global flow `ℝ → M → M`. - [ ] depends on: #21777 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-differential-geometry merge-conflict blocked-by-other-PR WIP 948/408 Mathlib/Algebra/Order/Group/Abs.lean,Mathlib/Analysis/Normed/Group/Basic.lean,Mathlib/Analysis/ODE/PicardLindelof.lean,Mathlib/Geometry/Manifold/IntegralCurve/Compact.lean,Mathlib/Geometry/Manifold/IntegralCurve/ExistUnique.lean,Mathlib/Order/Filter/Prod.lean,docs/1000.yaml,docs/undergrad.yaml 8 5 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
16-64919
16 days ago
16-64921
16 days ago
0-18
18 seconds
25057 mattrobball
author:mattrobball
test merge-conflict 23/12 Mathlib/Data/Finsupp/Defs.lean,Mathlib/RingTheory/AlgebraTower.lean,Mathlib/RingTheory/MvPowerSeries/Basic.lean 3 7 ['github-actions', 'leanprover-bot', 'leanprover-community-bot-assistant', 'mattrobball'] nobody
16-57280
16 days ago
16-57282
16 days ago
0-0
0 seconds
22073 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. --- - [ ] depends on: #21966 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta merge-conflict blocked-by-other-PR 983/1 Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Order.lean,Mathlib/Tactic/Order/CollectFacts.lean,Mathlib/Tactic/Order/Graph/Basic.lean,Mathlib/Tactic/Order/Graph/Tarjan.lean,Mathlib/Tactic/Order/Preprocessing.lean,MathlibTest/order.lean,scripts/noshake.json 9 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
16-28334
16 days ago
105-61166
3 months ago
0-32
32 seconds
20241 vasnesterov
author:vasnesterov
feat(Data/Seq): coinductive predicates for sequences * Introduce `All`, `Pairwise`, `AtLeastAsLongAs` predicates for sequences along with their coinductive principles and basic lemmas about them. * Prove `eq_of_bisim'` and `eq_of_bisim_strong` coinductive principles for equality. All of these "coinductive principles" are stated in the form as similar as possible to inductive principles. --- I also added `set_option linter.style.longFile 2000` in the beginning of `Seq.lean`, because I am not sure how to split this file. - [ ] depends on: #20160 This PR is necessary for a new tactic (#18486), which computes the asymptotics of real functions. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data merge-conflict blocked-by-other-PR 512/1 Mathlib/Data/Seq/Seq.lean 1 4 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
15-24552
15 days ago
15-24554
15 days ago
0-215
3 minutes
20818 artie2000
author:artie2000
feat(Algebra/Group/Even): Add missing lemmas * Make API for `IsSquare` / `Even` consistent between the "official" definition and equivalent ones * Add new lemma `exists_apply_eq_and_isSquare ` that's analogous to `IsSquare.map` --- - [x] depends on: #20558 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-algebra merge-conflict awaiting-author
label:t-algebra$
39/28 Mathlib/Algebra/Group/Even.lean,Mathlib/Data/Set/Basic.lean,Mathlib/Data/Set/Operations.lean 3 26 ['YaelDillies', 'alreadydone', 'artie2000', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'mergify'] nobody
15-24430
15 days ago
15-24431
15 days ago
0-3431
57 minutes
13026 BoltonBailey
author:BoltonBailey
feat: add `simp` lemma `coeff_eq_zero_of_not_mem_support` Adds the forward direction of `not_mem_support_iff` as a `simp` lemma. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra awaiting-CI merge-conflict help-wanted
label:t-algebra$
4/0 Mathlib/Algebra/MvPolynomial/Basic.lean 1 4 ['BoltonBailey', 'github-actions', 'grunweg', 'leanprover-community-bot-assistant'] nobody
15-22933
15 days ago
15-22935
15 days ago
0-0
0 seconds
22837 joneugster
author:joneugster
feat(Data/Set/Basic): add subset_iff and not_mem_subset_iff Add `Set.subset_iff` for consistent API with `Finset.subset_iff`. Add `Set.not_mem_subset_iff` and `Finset.not_mem_subset_iff`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-set-theory t-data merge-conflict 9/0 Mathlib/Data/Finset/Defs.lean,Mathlib/Data/Set/Basic.lean 2 4 ['Ruben-VandeVelde', 'github-actions', 'joneugster', 'leanprover-community-bot-assistant'] nobody
15-22167
15 days ago
15-22169
15 days ago
30-35190
30 days
23489 plp127
author:plp127
chore: fix recursors Replace motive with `motive` and other improvements. Will probably split this PR after fixing is done. 4013 recursors left --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP 4255/172 Mathlib/Algebra/EuclideanDomain/Basic.lean,Mathlib/Algebra/EuclideanDomain/Defs.lean,Mathlib/Algebra/Free.lean,Mathlib/Algebra/FreeMonoid/Basic.lean,Mathlib/Algebra/Group/Defs.lean,Mathlib/Algebra/Lie/BaseChange.lean,Mathlib/Algebra/Lie/IdealOperations.lean,Mathlib/Algebra/Lie/TraceForm.lean,Mathlib/Algebra/Order/Rearrangement.lean,Mathlib/Algebra/Ring/Subsemiring/Basic.lean,Mathlib/AlgebraicTopology/SimplexCategory/GeneratorsRelations/Basic.lean,Mathlib/Analysis/BoxIntegral/Partition/SubboxInduction.lean,Mathlib/CategoryTheory/Quotient.lean,Mathlib/Data/Fin/Basic.lean,Mathlib/Data/Fin/Tuple/Basic.lean,Mathlib/Data/Fin/Tuple/BubbleSortInduction.lean,Mathlib/Data/Fin/Tuple/NatAntidiagonal.lean,Mathlib/Data/FinEnum/Option.lean,Mathlib/Data/Finset/Max.lean,Mathlib/Data/Fintype/CardEmbedding.lean,Mathlib/Data/Fintype/Option.lean,Mathlib/Data/NNRat/Defs.lean,Mathlib/Data/Nat/BinaryRec.lean,Mathlib/Data/PFun.lean,Mathlib/Data/PFunctor/Multivariate/W.lean,Mathlib/Data/Quot.lean,Mathlib/Data/Sym/Sym2.lean,Mathlib/GroupTheory/Congruence/Defs.lean,Mathlib/GroupTheory/Coprod/Basic.lean,Mathlib/GroupTheory/Coset/Defs.lean,Mathlib/GroupTheory/Coxeter/Basic.lean,Mathlib/LinearAlgebra/Span/Defs.lean,Mathlib/LinearAlgebra/TensorProduct/Tower.lean,Mathlib/NumberTheory/LSeries/HurwitzZetaEven.lean,Mathlib/NumberTheory/LSeries/HurwitzZetaOdd.lean,Mathlib/Order/DirectedInverseSystem.lean,Mathlib/RingTheory/AdicCompletion/Basic.lean,Mathlib/SetTheory/Cardinal/Defs.lean,Mathlib/SetTheory/PGame/Algebra.lean,done.csv,print.lean,working.csv 42 3 ['github-actions', 'leanprover-community-bot-assistant'] nobody
15-21648
15 days ago
15-21649
15 days ago
0-0
0 seconds
24096 plp127
author:plp127
feat(Topology): Completely Regular Space iff Uniformizable Proves that `CompletelyRegularSpace`s are uniformizable and that `UniformSpace`s are completely regular. --- - [x] depends on: #24179 - [ ] depends on: #24173 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology merge-conflict blocked-by-other-PR 374/31 Mathlib.lean,Mathlib/Topology/Bases.lean,Mathlib/Topology/UniformSpace/Basic.lean,Mathlib/Topology/UniformSpace/Defs.lean,Mathlib/Topology/UniformSpace/Uniformizable.lean,Mathlib/Topology/UrysohnsLemma.lean 6 9 ['alreadydone', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'plp127'] nobody
15-21524
15 days ago
15-21526
15 days ago
2-6687
2 days
24100 eric-wieser
author:eric-wieser
feat: restore some explicit binders from Lean 3 Part of #24099 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) tech debt merge-conflict awaiting-author 39/42 Mathlib/Data/FinEnum.lean,Mathlib/FieldTheory/Galois/Profinite.lean,Mathlib/Topology/Bases.lean,Mathlib/Topology/Compactness/CompactlyGeneratedSpace.lean,Mathlib/Topology/MetricSpace/IsometricSMul.lean,Mathlib/Topology/Metrizable/CompletelyMetrizable.lean,Mathlib/Topology/Metrizable/Uniformity.lean,Mathlib/Topology/Order.lean,Mathlib/Topology/Order/LowerUpperTopology.lean,Mathlib/Topology/UniformSpace/UniformEmbedding.lean 10 3 ['github-actions', 'grunweg', 'leanprover-community-bot-assistant'] nobody
15-21523
15 days ago
15-21525
15 days ago
34-33204
34 days
25143 chrisflav
author:chrisflav
feat(RingTheory): smooth algebras have smooth Noetherian models Co-authored by: Judith Ludwig --- - [ ] depends on: #24794 - [ ] depends on: #25138 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict blocked-by-other-PR
label:t-algebra$
596/45 Mathlib.lean,Mathlib/Algebra/Algebra/Subalgebra/Basic.lean,Mathlib/Algebra/Algebra/Subalgebra/Tower.lean,Mathlib/Algebra/Algebra/Tower.lean,Mathlib/Algebra/MvPolynomial/Basic.lean,Mathlib/Algebra/MvPolynomial/Eval.lean,Mathlib/RingTheory/AlgebraicIndependent/Transcendental.lean,Mathlib/RingTheory/Extension/Presentation/Basic.lean,Mathlib/RingTheory/Extension/Presentation/Core.lean,Mathlib/RingTheory/FinitePresentation.lean,Mathlib/RingTheory/FiniteType.lean,Mathlib/RingTheory/Ideal/Cotangent.lean,Mathlib/RingTheory/Ideal/Maps.lean,Mathlib/RingTheory/Ideal/Quotient/Operations.lean,Mathlib/RingTheory/MvPolynomial/Homogeneous.lean,Mathlib/RingTheory/Smooth/Basic.lean,Mathlib/RingTheory/Smooth/Kaehler.lean,Mathlib/RingTheory/Smooth/NoetherianDescent.lean,Mathlib/RingTheory/Spectrum/Prime/ChevalleyComplexity.lean,Mathlib/RingTheory/TensorProduct/MvPolynomial.lean,Mathlib/RingTheory/Unramified/Basic.lean 21 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
15-21147
15 days ago
15-21149
15 days ago
0-713
11 minutes
21476 grunweg
author:grunweg
feat(lint-style): enable running on downstream projects Enable lint-style to run on downstream projects, by making the following modifications: - allow passing an explicit list of libraries to lint: if nothing is passed, it lints `Mathlib`, `Archive` and `Counterexamples` (as before); otherwise, it lints precisely the passed modules - only check init imports, undocumented scripts and the errors from `lint-style.py` when linting Mathlib - make the style exceptions file configurable and optional: using the `nolints-file` flag, the exceptions file can be configured. If the flag is omitted, we try to find a file at `scripts/nolints-style.txt` --- and otherwise proceed with no style exceptions. This means mathlib can continue unchanged, and downstream projects can either add an explicit exceptions file, or proceed without any exceptions. After this PR, one should be able to run lint-style on a downstream project by `lake exe lint-style ProjectName`. Prompted by [this zulip discussion](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/lint-style.20for.20downstream.20libraries). --- - [ ] depends on: #24570 - [ ] depends on: #24953 (I did not test the last part.) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-linter merge-conflict 58/19 Mathlib/Tactic/Linter/TextBased.lean,scripts/lint-style.lean 2 19 ['Vierkantor', 'adomani', 'github-actions', 'grunweg', 'joneugster', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] joneugster
assignee:joneugster
14-27655
14 days ago
14-27658
14 days ago
43-17409
43 days
24163 urkud
author:urkud
refactor(TangentCone): redefine for TVS --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis merge-conflict 421/284 Mathlib/Analysis/Calculus/FDeriv/Basic.lean,Mathlib/Analysis/Calculus/TangentCone.lean,Mathlib/Topology/Algebra/ConstMulAction.lean 3 4 ['github-actions', 'leanprover-community-bot-assistant'] nobody
13-59372
13 days ago
13-59373
13 days ago
0-0
0 seconds
23915 joelriou
author:joelriou
feat(CategoryTheory): deriving functors using a right derivability structure We develop the API for derived functors following the existence theorem obtained in #22508. If `Φ` is a localizer morphism, we introduce a predicate `Φ.Derives F` for a functor `F` saying that `Φ.functor ⋙ F` inverts the given class of morphisms, and in case `Φ` is a right derivability structure, we show that `F` admits a right derived functor, and we obtain a recognition lemma for this derived functor. (In the future, this will be applied to the injective/projective/flat derivability structures.) --- - [ ] depends on: #22508 - [ ] depends on: #22474 - [ ] depends on: #22490 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory merge-conflict blocked-by-other-PR WIP 599/10 Mathlib.lean,Mathlib/CategoryTheory/Functor/Derived/PointwiseRightDerived.lean,Mathlib/CategoryTheory/Functor/Derived/RightDerived.lean,Mathlib/CategoryTheory/Functor/KanExtension/Pointwise.lean,Mathlib/CategoryTheory/Iso.lean,Mathlib/CategoryTheory/Limits/Final.lean,Mathlib/CategoryTheory/Limits/HasLimits.lean,Mathlib/CategoryTheory/Limits/Opposites.lean,Mathlib/CategoryTheory/Limits/Shapes/Products.lean,Mathlib/CategoryTheory/Localization/DerivabilityStructure/Basic.lean,Mathlib/CategoryTheory/Localization/DerivabilityStructure/Derives.lean,Mathlib/CategoryTheory/Localization/DerivabilityStructure/PointwiseRightDerived.lean 12 4 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
13-46953
13 days ago
28-83619
28 days ago
0-0
0 seconds
22508 joelriou
author:joelriou
feat(CategoryTheory): existence of right derived functors using derivability structures In this PR, we formalize an existence theorem for right derived functors which appeared in the article *Structures de dérivabilité* by Bruno Kahn and Georges Maltsiniotis, Adv. Math. 218 (2008). --- - [ ] depends on: #22474 - [ ] depends on: #22490 - [x] depends on: #22514 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory merge-conflict blocked-by-other-PR WIP 480/9 Mathlib.lean,Mathlib/CategoryTheory/Functor/Derived/PointwiseRightDerived.lean,Mathlib/CategoryTheory/Functor/KanExtension/Pointwise.lean,Mathlib/CategoryTheory/Iso.lean,Mathlib/CategoryTheory/Limits/Final.lean,Mathlib/CategoryTheory/Limits/HasLimits.lean,Mathlib/CategoryTheory/Limits/Opposites.lean,Mathlib/CategoryTheory/Limits/Shapes/Products.lean,Mathlib/CategoryTheory/Localization/DerivabilityStructure/Basic.lean,Mathlib/CategoryTheory/Localization/DerivabilityStructure/PointwiseRightDerived.lean 10 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
13-46915
13 days ago
42-40479
1 month ago
0-0
0 seconds
21127 jt496
author:jt496
feat(Combinatorics/SimpleGraph): the Andrásfai–Erdős–Sós theorem Co-authored-by: Lian Tattersall --- This is a draft version of our formalisation of the Andrásfai–Erdős–Sós theorem. We intend to split this into smaller pieces for review/revision. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-combinatorics merge-conflict WIP 487/0 Mathlib.lean,Mathlib/Combinatorics/SimpleGraph/FiveWheelLike.lean 2 2 ['github-actions', 'leanprover-community-bot-assistant'] nobody
13-34776
13 days ago
13-34778
13 days ago
0-0
0 seconds
21844 smmercuri
author:smmercuri
feat: the ring of integers of a `ℤₘ₀`-valued field is compact whenever it is a DVR and the residue field is finite --- - [ ] depends on: #21162 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-algebra merge-conflict blocked-by-other-PR
label:t-algebra$
166/3 Mathlib.lean,Mathlib/Algebra/Order/GroupWithZero/Canonical.lean,Mathlib/RingTheory/DedekindDomain/AdicValuation.lean,Mathlib/RingTheory/Ideal/Quotient/Basic.lean,Mathlib/Topology/Algebra/Valued/LocallyCompact.lean,Mathlib/Topology/Algebra/Valued/ValuationTopology.lean,Mathlib/Topology/Algebra/Valued/WithZeroMulInt.lean 7 4 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
13-32888
13 days ago
13-32889
13 days ago
0-879
14 minutes
23349 BGuillemet
author:BGuillemet
feat: add LocallyLipschitzOn.lipschitzOnWith_of_isCompact and two small lemmas about Lipschitz functions Main feat (in Mathlib/Topology/EMetricSpace/Basic.lean): if a function `f` from an extended pseudometric space to a pseudometric space is locally Lipschitz on a compact subset `s`, then `f` is Lipschitz on `s`. The theorem is true only when the codomain of `f` is a pseudometric space, so it needs imports from Mathlib/Topology/MetricSpace. Other small feat (in Mathlib/Analysis/Calculus/ContDiff/RCLike.lean): a function that is continuously differentiable on an open subset is locally Lipschitz on this subset. --- - [ ] depends on: #22890 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import new-contributor t-topology merge-conflict 59/4 Mathlib/Analysis/Calculus/ContDiff/RCLike.lean,Mathlib/Topology/EMetricSpace/Lipschitz.lean 2 4 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] PatrickMassot
assignee:PatrickMassot
13-9385
13 days ago
13-9387
13 days ago
35-30364
35 days
23333 mariainesdff
author:mariainesdff
feat(Analysis.Normed.Unbundled.SpectralNormUnique): prove unique extension theorem Let `K` be a field complete with respect to a nontrivial nonarchimedean multiplicative norm and `L/K` be an algebraic extension. We show that the spectral norm on `L` is a nonarchimedean multiplicative norm, and any power-multiplicative `K`-algebra norm on `L` coincides with the spectral norm. More over, if `L/K` is finite, then `L` is a complete space. This result is [S. Bosch, U. Güntzer, R. Remmert,*Non-Archimedean Analysis* (Theorem 3.2.4/2)][bosch-guntzer-remmert]. --- - [ ] depends on: #23301 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-analysis t-number-theory merge-conflict 1487/3 Mathlib.lean,Mathlib/Algebra/Order/BigOperators/Ring/Finset.lean,Mathlib/Algebra/Order/BigOperators/Ring/Multiset.lean,Mathlib/Algebra/Polynomial/Basic.lean,Mathlib/Algebra/Polynomial/BigOperators.lean,Mathlib/Algebra/Polynomial/Lifts.lean,Mathlib/Algebra/Polynomial/RingDivision.lean,Mathlib/Algebra/Polynomial/Splits.lean,Mathlib/Analysis/Normed/Unbundled/AlgNormOfGalois.lean,Mathlib/Analysis/Normed/Unbundled/RingSeminorm.lean,Mathlib/Analysis/Normed/Unbundled/SpectralNorm.lean,Mathlib/Analysis/Normed/Unbundled/SpectralNormUnique.lean,Mathlib/Data/Finset/Max.lean,Mathlib/Data/List/MinMax.lean,Mathlib/Data/NNReal/Basic.lean,Mathlib/Data/Real/IsNonarchimedean.lean,Mathlib/Data/Real/Pointwise.lean,Mathlib/FieldTheory/IntermediateField/Adjoin/Basic.lean,Mathlib/FieldTheory/IsAlgClosed/AlgebraicClosure.lean,Mathlib/Order/ConditionallyCompleteLattice/Finset.lean,Mathlib/Order/ConditionallyCompleteLattice/Indexed.lean 21 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
12-77352
12 days ago
12-77354
12 days ago
0-0
0 seconds
22724 peabrainiac
author:peabrainiac
feat(Geometry/Diffeology): diffeologies generated from sets of plots Introduces diffeologies generated from sets of plots, shows that this defines a Galois insertion, and concludes that the diffeologies on a type from a complete lattice. --- - [ ] depends on: #21969 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-differential-geometry merge-conflict blocked-by-other-PR 631/0 Mathlib.lean,Mathlib/Geometry/Diffeology/Basic.lean,docs/references.bib,scripts/noshake.json 4 4 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
12-46732
12 days ago
12-46734
12 days ago
0-518
8 minutes
8949 sebzim4500
author:sebzim4500
Add `by_approx` tactic for proving real inequalities using rational approximation feat: Add `by_approx` tactic for proving real inequalities by finding rational approximations --- ```lean example : |sqrt 2 - 1.414| < 0.001 := by by_approx ``` This is a work in progress, the code is messy and the tactic is often very slow. It also depends on some other PRs that haven't been merged yet. It currently supports basic operations (`+`, `-`, `*`, `/`, `abs`) and has approximation extensions for `sqrt` and `exp`. - [ ] depends on: #8167 - [x] depends on: #8832 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta merge-conflict modifies-tactic-syntax blocked-by-other-PR 1670/3 Mathlib.lean,Mathlib/Data/Int/ModEq.lean,Mathlib/Tactic.lean,Mathlib/Tactic/ByApprox.lean,Mathlib/Tactic/ByApprox/Basic.lean,Mathlib/Tactic/ByApprox/Core.lean,Mathlib/Tactic/ByApprox/Exp.lean,Mathlib/Tactic/ByApprox/Lemmas.lean,Mathlib/Tactic/ByApprox/Test.lean,Mathlib/Tactic/ByApprox/Util.lean,Mathlib/Tactic/GCongr/Core.lean,Mathlib/Tactic/GRW.lean,Mathlib/Tactic/GRW/Core.lean,Mathlib/Tactic/GRW/Lemmas.lean,Mathlib/Tactic/NormNum/NatFactorial.lean,test/ByApprox.lean,test/GRW.lean,test/norm_num_ext.lean 18 1 ['leanprover-community-mathlib4-bot'] nobody
12-20079
12 days ago
377-45989
1 year ago
0-0
0 seconds
20380 mans0954
author:mans0954
feature(Analysis/NormedSpace/MStructure): The component projections on WithLp 1 (α × β) are L-projections The component idempotents on `WithLp 1 (α × β)` are L-projections (It's possible to formulate a definition of an `Lᵖ`-projection so that this result would hold for `(p : ℝ≥0∞)` but this would introduce considerable extra complexity so is not considered in this PR.) --- - [ ] depends on: #21899 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-analysis merge-conflict awaiting-author 20/1 Mathlib.lean,Mathlib/Analysis/Normed/Lp/MStructure.lean,Mathlib/Analysis/Normed/Lp/ProdLp.lean 3 26 ['eric-wieser', 'github-actions', 'j-loreaux', 'leanprover-community-bot-assistant', 'mans0954', 'mathlib4-dependent-issues-bot'] nobody
12-11416
12 days ago
12-11418
12 days ago
43-49391
43 days
23767 grunweg
author:grunweg
refactor: make library notes a definition Make library notes a definition of `Unit` type, whose doc-string is the note's content. As a consequence, - doc-gen will display all library notes without any custom logic, - library notes are shown upon hover (via the use of the doc-string), - go do definition for library notes is easy Automate this using a macro, which also enforces that all library notes are inside the Mathlib.LibraryNote namespace. *Temporarily*, we use the `library_note2` name; if/when the batteries version is changed, we can reclaim the original name. This PR does not address how to *refer* to library notes nicely (in a way that is shown in the documentation, checked for typos, with sufficient imports ensured etc.). That is left to a future PR. This is proposal 2a from this [zulip discussion]([#mathlib4 > library notes @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/library.20notes/near/510614740)) ------------ Open questions/TODOs: - should this go in batteries instead? can the old definition just be overwritten? - otherwise, what's the best place for the `LibraryNote` definition? A single file just for this feels overkill; I put it in Mathlib.Tactic.Basic for now. I could use Mathlib.Init, of course (but that might be excessive) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-meta merge-conflict 48/48 Archive/Imo/Imo2019Q2.lean,Mathlib/Algebra/BigOperators/Group/Finset/Defs.lean,Mathlib/Algebra/Category/Ring/Limits.lean,Mathlib/Algebra/Group/Action/Defs.lean,Mathlib/Algebra/Group/Conj.lean,Mathlib/Algebra/Group/Defs.lean,Mathlib/Algebra/Group/Hom/Defs.lean,Mathlib/Algebra/Group/Pointwise/Set/Basic.lean,Mathlib/Algebra/Group/Pointwise/Set/Scalar.lean,Mathlib/Algebra/Group/Submonoid/Operations.lean,Mathlib/Algebra/HierarchyDesign.lean,Mathlib/Algebra/Order/Hom/Basic.lean,Mathlib/Analysis/CStarAlgebra/ContinuousFunctionalCalculus/Note.lean,Mathlib/Analysis/RCLike/Lemmas.lean,Mathlib/CategoryTheory/Category/Basic.lean,Mathlib/Data/NNRat/Defs.lean,Mathlib/Data/Nat/Cast/Defs.lean,Mathlib/Data/Nat/Init.lean,Mathlib/Geometry/Manifold/Algebra/Monoid.lean,Mathlib/Geometry/Manifold/ChartedSpace.lean,Mathlib/Logic/Basic.lean,Mathlib/Tactic/Basic.lean,Mathlib/Tactic/NormNum/Basic.lean,Mathlib/Tactic/Simps/Basic.lean,Mathlib/Topology/Algebra/Nonarchimedean/Bases.lean,Mathlib/Topology/Continuous.lean 26 9 ['adomani', 'github-actions', 'grunweg', 'leanprover-community-bot-assistant'] nobody
11-22480
11 days ago
11-22482
11 days ago
51-69759
51 days
25141 eric-wieser
author:eric-wieser
feat: basis for multilinear maps This attempts to tease an intermediate result out of #11155, which lets us show that multilinear maps are free even if their codomain is not finite. I guess this continues from https://github.com/leanprover-community/mathlib3/pull/10504 and https://github.com/leanprover-community/mathlib3/pull/14199. --- - [ ] depends on: #11155 - [ ] depends on: #25142 - [ ] depends on: #25169 - [ ] depends on: #25166 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-algebra merge-conflict blocked-by-other-PR
label:t-algebra$
507/45 Mathlib.lean,Mathlib/LinearAlgebra/DFinsupp.lean,Mathlib/LinearAlgebra/DFinsupp/PiTensorProduct.lean,Mathlib/LinearAlgebra/DirectSum/Finsupp.lean,Mathlib/LinearAlgebra/DirectSum/PiTensorProduct.lean,Mathlib/LinearAlgebra/Multilinear/Basic.lean,Mathlib/LinearAlgebra/Multilinear/Basis.lean,Mathlib/LinearAlgebra/Multilinear/DFinsupp.lean,Mathlib/LinearAlgebra/Multilinear/DirectSum.lean,Mathlib/LinearAlgebra/Multilinear/FiniteDimensional.lean,Mathlib/LinearAlgebra/Multilinear/Pi.lean 11 4 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
11-12772
11 days ago
11-12773
11 days ago
0-0
0 seconds
12438 jjaassoonn
author:jjaassoonn
feat: some APIs for flat modules Need horseshoe lemma --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory merge-conflict WIP 1674/3 Mathlib.lean,Mathlib/Algebra/Category/ModuleCat/Monoidal/Basic.lean,Mathlib/Algebra/Category/ModuleCat/Monoidal/Symmetric.lean,Mathlib/Algebra/Exact.lean,Mathlib/CategoryTheory/Abelian/Basic.lean,Mathlib/CategoryTheory/Abelian/DiagramLemmas/Horseshoe.lean,Mathlib/CategoryTheory/Abelian/LeftDerived.lean,Mathlib/RingTheory/Flat/Basic.lean 8 21 ['erdOne', 'github-actions', 'jjaassoonn', 'joelriou'] nobody
8-22011
8 days ago
394-39428
1 year ago
0-0
0 seconds
23282 joelriou
author:joelriou
feat(CategoryTheory): monomorphisms in Type are stable under transfinite compositions `monomorphisms (Type u)` is stable under cobase change, filtered colimits and transfinite compositions. (The file `CategoryTheory.Types` is also moved to `CategoryTheory.Types.Basic`.) (This is extended to presheaves of types in #23298.) --- - [x] depends on: #24773 - [ ] depends on: #24777 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-category-theory merge-conflict blocked-by-other-PR WIP 739/642 Mathlib.lean,Mathlib/CategoryTheory/Abelian/GrothendieckAxioms/Colim.lean,Mathlib/CategoryTheory/Abelian/GrothendieckCategory/EnoughInjectives.lean,Mathlib/CategoryTheory/Abelian/GrothendieckCategory/Monomorphisms.lean,Mathlib/CategoryTheory/Category/Cat.lean,Mathlib/CategoryTheory/Category/RelCat.lean,Mathlib/CategoryTheory/ConcreteCategory/Basic.lean,Mathlib/CategoryTheory/ConcreteCategory/EpiMono.lean,Mathlib/CategoryTheory/Core.lean,Mathlib/CategoryTheory/Functor/Hom.lean,Mathlib/CategoryTheory/IsomorphismClasses.lean,Mathlib/CategoryTheory/Limits/Types/Shapes.lean,Mathlib/CategoryTheory/Localization/FiniteProducts.lean,Mathlib/CategoryTheory/Monad/Types.lean,Mathlib/CategoryTheory/MorphismProperty/FunctorCategory.lean,Mathlib/CategoryTheory/MorphismProperty/LiftingProperty.lean,Mathlib/CategoryTheory/MorphismProperty/Limits.lean,Mathlib/CategoryTheory/MorphismProperty/TransfiniteComposition.lean,Mathlib/CategoryTheory/SmallObject/IsCardinalForSmallObjectArgument.lean,Mathlib/CategoryTheory/SmallObject/WellOrderInductionData.lean,Mathlib/CategoryTheory/Subobject/Types.lean,Mathlib/CategoryTheory/Types.lean,Mathlib/CategoryTheory/Types/Basic.lean,Mathlib/CategoryTheory/Types/Monomorphisms.lean,Mathlib/CategoryTheory/UnivLE.lean,Mathlib/Control/Fold.lean,Mathlib/Data/Set/FunctorToTypes.lean 27 14 ['callesonne', 'erdOne', 'github-actions', 'joelriou', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
8-14275
8 days ago
27-14063
27 days ago
45-69656
45 days
24409 urkud
author:urkud
chore(*): fix `nmem` vs `not_mem` names --- There are some missing/buggy deprecations, I'm going to fix them later today or tomorrow. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-zulip tech debt merge-conflict delegated awaiting-author 317/176 Mathlib/Algebra/BigOperators/Finprod.lean,Mathlib/Algebra/BigOperators/Group/Finset/Lemmas.lean,Mathlib/Algebra/Group/Indicator.lean,Mathlib/Algebra/Group/Support.lean,Mathlib/Algebra/GroupWithZero/NonZeroDivisors.lean,Mathlib/Algebra/Order/Group/Indicator.lean,Mathlib/Algebra/Polynomial/AlgebraMap.lean,Mathlib/Algebra/Polynomial/Degree/Operations.lean,Mathlib/Analysis/Calculus/BumpFunction/Basic.lean,Mathlib/Analysis/Calculus/DSlope.lean,Mathlib/Analysis/Calculus/Deriv/Basic.lean,Mathlib/Analysis/Calculus/Deriv/Support.lean,Mathlib/Analysis/Calculus/FDeriv/Basic.lean,Mathlib/Analysis/Calculus/Rademacher.lean,Mathlib/Analysis/Complex/RemovableSingularity.lean,Mathlib/Analysis/Convex/Cone/InnerDual.lean,Mathlib/Analysis/Convex/Cone/Proper.lean,Mathlib/Analysis/Convolution.lean,Mathlib/Analysis/Distribution/AEEqOfIntegralContDiff.lean,Mathlib/Data/LocallyFinsupp.lean,Mathlib/Data/Set/Basic.lean,Mathlib/Data/Set/Insert.lean,Mathlib/Dynamics/Ergodic/Conservative.lean,Mathlib/Dynamics/Ergodic/Ergodic.lean,Mathlib/Dynamics/Ergodic/Function.lean,Mathlib/Dynamics/PeriodicPts/Defs.lean,Mathlib/Geometry/Manifold/ContMDiff/Basic.lean,Mathlib/Geometry/Manifold/PartitionOfUnity.lean,Mathlib/GroupTheory/CosetCover.lean,Mathlib/LinearAlgebra/Dual/Lemmas.lean,Mathlib/LinearAlgebra/FreeModule/PID.lean,Mathlib/LinearAlgebra/PID.lean,Mathlib/LinearAlgebra/RootSystem/Base.lean,Mathlib/LinearAlgebra/RootSystem/Finite/Lemmas.lean,Mathlib/MeasureTheory/Function/ContinuousMapDense.lean,Mathlib/MeasureTheory/Function/ConvergenceInMeasure.lean,Mathlib/MeasureTheory/Function/L2Space.lean,Mathlib/MeasureTheory/Function/LocallyIntegrable.lean,Mathlib/MeasureTheory/Function/LpSpace/Indicator.lean,Mathlib/MeasureTheory/Integral/Average.lean,Mathlib/MeasureTheory/Integral/Bochner/Set.lean,Mathlib/MeasureTheory/Integral/Layercake.lean,Mathlib/MeasureTheory/Integral/Lebesgue/Add.lean,Mathlib/MeasureTheory/Integral/Lebesgue/Basic.lean,Mathlib/MeasureTheory/Integral/RieszMarkovKakutani/Basic.lean,Mathlib/MeasureTheory/Integral/RieszMarkovKakutani/Real.lean,Mathlib/MeasureTheory/Measure/AbsolutelyContinuous.lean,Mathlib/MeasureTheory/Measure/AddContent.lean,Mathlib/MeasureTheory/Measure/DiracProba.lean,Mathlib/MeasureTheory/Measure/Haar/Unique.lean,Mathlib/MeasureTheory/Measure/Restrict.lean,Mathlib/MeasureTheory/Measure/WithDensity.lean,Mathlib/MeasureTheory/OuterMeasure/AE.lean,Mathlib/MeasureTheory/SetSemiring.lean,Mathlib/Order/Filter/AtTopBot/CountablyGenerated.lean,Mathlib/Order/Filter/Cocardinal.lean,Mathlib/Order/Filter/Cofinite.lean,Mathlib/Order/Filter/Tendsto.lean,Mathlib/Order/Filter/Ultrafilter/Basic.lean,Mathlib/Probability/Distributions/Uniform.lean,Mathlib/Probability/Kernel/Basic.lean,Mathlib/Probability/Kernel/Composition/MeasureCompProd.lean,Mathlib/RingTheory/AdicCompletion/LocalRing.lean,Mathlib/RingTheory/Ideal/Maximal.lean,Mathlib/RingTheory/LaurentSeries.lean,Mathlib/RingTheory/MvPolynomial/Symmetric/NewtonIdentities.lean,Mathlib/RingTheory/MvPowerSeries/NoZeroDivisors.lean,Mathlib/RingTheory/Spectrum/Maximal/Localization.lean,Mathlib/RingTheory/Spectrum/Prime/RingHom.lean,Mathlib/RingTheory/Spectrum/Prime/Topology.lean,Mathlib/Topology/Algebra/InfiniteSum/Group.lean,Mathlib/Topology/Algebra/Module/Cardinality.lean,Mathlib/Topology/Algebra/Support.lean,Mathlib/Topology/Bases.lean,Mathlib/Topology/ContinuousMap/BoundedCompactlySupported.lean,Mathlib/Topology/Order/Basic.lean,Mathlib/Topology/UrysohnsLemma.lean 77 4 ['b-mehta', 'github-actions', 'jcommelin', 'leanprover-community-bot-assistant', 'mathlib-bors'] nobody
7-49043
7 days ago
7-49043
7 days ago
0-55045
15 hours
24596 joelriou
author:joelriou
feat(Algebra/Homology): the derived category of a linear abelian category is linear --- - [ ] depends on: #24191 - [ ] depends on: #24567 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory merge-conflict blocked-by-other-PR WIP 397/189 Mathlib.lean,Mathlib/Algebra/Homology/DerivedCategory/Basic.lean,Mathlib/Algebra/Homology/DerivedCategory/Linear.lean,Mathlib/Algebra/Homology/HomotopyCategory/Shift.lean,Mathlib/Algebra/Homology/HomotopyCategory/SingleFunctors.lean,Mathlib/CategoryTheory/ObjectProperty/ContainsZero.lean,Mathlib/CategoryTheory/ObjectProperty/Shift.lean,Mathlib/CategoryTheory/Shift/Linear.lean,Mathlib/CategoryTheory/Triangulated/HomologicalFunctor.lean,Mathlib/CategoryTheory/Triangulated/Subcategory.lean 10 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
7-45066
7 days ago
28-7770
28 days ago
0-0
0 seconds
23730 faenuccio
author:faenuccio
feat: define valued local fields Co-authored by: @mariainesdff --- - [x] depends on: #23725 - [x] depends on: #23726 - [ ] depends on: #23727 large-import t-algebra t-number-theory merge-conflict blocked-by-other-PR
label:t-algebra$
122/21 Mathlib.lean,Mathlib/NumberTheory/LocalField/Valued.lean,Mathlib/RingTheory/Valuation/Discrete/Basic.lean,docs/references.bib 4 11 ['faenuccio', 'github-actions', 'kbuzzard', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
7-40993
7 days ago
28-8020
28 days ago
2-9769
2 days
21129 chrisflav
author:chrisflav
perf(RingTheory/Kaehler/JacobiZariski): reorder universe variables Naming of universe variables has an impact on universe unification. It seems to matter that the universe variables of `R`, `S` and `T` appear before the universe variables of the generators in alphabetical order. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) performance-hack t-algebra merge-conflict
label:t-algebra$
18/20 Mathlib/RingTheory/Kaehler/JacobiZariski.lean 1 38 ['chrisflav', 'erdOne', 'github-actions', 'grunweg', 'kbuzzard', 'leanprover-bot', 'leanprover-community-bot-assistant', 'mattrobball'] nobody
7-24653
7 days ago
7-24655
7 days ago
125-81208
125 days
24396 JovanGerb
author:JovanGerb
feat(Order/Defs): refactor in preparation of `to_dual` attribute When the `to_dual` attribute lands in Mathlib, we will tag many lemmas about order with this tag, which will automatically give us the dual statements. This PR prepares for this by - moving dual declarations closer together - replacing occurrences of `>` and `≥` with `<` and `≤` - consistently applying a new naming convention that helps us to name dual lemmas: we use the keywords `ge` and `gt` in place of `le` and `lt` to indicate that the same pair `a, b` in `a < b` is in the opposite order to the order in which it appeared the first time. - when we have to disambiguate the order of the argument to `<` or `≤`, we sometimes use `gt` or `ge` instead of `lt` or `le`. We also use this to get rid of many primed lemma names. This is a copy of #24376, but it doesn't remove the old lemma names, so doesn't require making changes in >500 files. deprecating these lemmas will be left to a future PR. [#mathlib4 > naming convention for ≤ and <](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/naming.20convention.20for.20.E2.89.A4.20and.20.3C) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-zulip t-order merge-conflict 248/230 Mathlib/Algebra/Order/CauSeq/Basic.lean,Mathlib/Algebra/Order/Ring/Unbundled/Rat.lean,Mathlib/Algebra/Polynomial/Degree/Domain.lean,Mathlib/Algebra/Tropical/Basic.lean,Mathlib/Analysis/SpecialFunctions/Pow/Continuity.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Arctan.lean,Mathlib/Computability/TuringMachine.lean,Mathlib/Data/Bool/Basic.lean,Mathlib/Data/Char.lean,Mathlib/Data/Complex/Order.lean,Mathlib/Data/ENat/Basic.lean,Mathlib/Data/Int/Order/Basic.lean,Mathlib/Data/Nat/Basic.lean,Mathlib/Data/Nat/Factorization/Defs.lean,Mathlib/Data/Nat/Find.lean,Mathlib/Data/Nat/PartENat.lean,Mathlib/Data/Num/Lemmas.lean,Mathlib/Data/Num/ZNum.lean,Mathlib/Data/PSigma/Order.lean,Mathlib/Data/Prod/Lex.lean,Mathlib/Data/Real/Basic.lean,Mathlib/Data/Setoid/Basic.lean,Mathlib/Data/Setoid/Partition.lean,Mathlib/Data/Sigma/Order.lean,Mathlib/Data/String/Basic.lean,Mathlib/Data/Sum/Order.lean,Mathlib/GroupTheory/MonoidLocalization/Order.lean,Mathlib/NumberTheory/Zsqrtd/Basic.lean,Mathlib/Order/Antisymmetrization.lean,Mathlib/Order/Basic.lean,Mathlib/Order/Booleanisation.lean,Mathlib/Order/Defs/LinearOrder.lean,Mathlib/Order/Defs/PartialOrder.lean,Mathlib/Order/RelClasses.lean,Mathlib/Order/WithBot.lean,Mathlib/Probability/Martingale/Upcrossing.lean,Mathlib/RingTheory/UniqueFactorizationDomain/Multiplicity.lean,Mathlib/SetTheory/Game/Basic.lean,Mathlib/SetTheory/Ordinal/Basic.lean,Mathlib/SetTheory/Ordinal/Notation.lean,Mathlib/SetTheory/Surreal/Basic.lean,Mathlib/Tactic/Linarith/Frontend.lean,MathlibTest/linarith.lean 43 5 ['JovanGerb', 'bryangingechen', 'github-actions', 'leanprover-community-bot-assistant'] bryangingechen
assignee:bryangingechen
7-11145
7 days ago
7-11147
7 days ago
5-75236
5 days
25138 chrisflav
author:chrisflav
chore(RingTheory): remove unnecessary `toRingHom` coercions --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict
label:t-algebra$
32/40 Mathlib/RingTheory/Extension/Presentation/Basic.lean,Mathlib/RingTheory/FinitePresentation.lean,Mathlib/RingTheory/Ideal/Cotangent.lean,Mathlib/RingTheory/Ideal/Maps.lean,Mathlib/RingTheory/Ideal/Quotient/Operations.lean,Mathlib/RingTheory/Smooth/Basic.lean,Mathlib/RingTheory/Smooth/Kaehler.lean,Mathlib/RingTheory/Spectrum/Prime/ChevalleyComplexity.lean,Mathlib/RingTheory/Unramified/Basic.lean 9 5 ['chrisflav', 'erdOne', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant'] nobody
7-10781
7 days ago
7-10783
7 days ago
9-64502
9 days
24965 erdOne
author:erdOne
refactor: Make `IsLocalHom` take unbundled map --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) maintainer-merge t-algebra merge-conflict awaiting-author
label:t-algebra$
16/7 Mathlib/Algebra/Group/Units/Hom.lean,Mathlib/AlgebraicGeometry/Scheme.lean,Mathlib/Geometry/RingedSpace/LocallyRingedSpace.lean,Mathlib/Geometry/RingedSpace/LocallyRingedSpace/HasColimits.lean,Mathlib/Geometry/RingedSpace/OpenImmersion.lean 5 6 ['alreadydone', 'erdOne', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant'] nobody
6-62766
6 days ago
6-62767
6 days ago
10-26015
10 days
8740 digama0
author:digama0
fix: improve `recall` impl / error reporting Simplifies the implementation of `recall`, fixing a bug [reported on Zulip](https://leanprover.zulipchat.com/#narrow/stream/113488-general/topic/.60recall.60.20strangeness/near/405076713) and also eliminating a use of `open private`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-CI t-meta merge-conflict awaiting-author 27/39 Mathlib/Tactic/Recall.lean 1 2 ['github-actions', 'leanprover-community-bot-assistant'] nobody
6-39272
6 days ago
6-39274
6 days ago
0-0
0 seconds
21182 joneugster
author:joneugster
fix(Util/CountHeartbeats): move elaboration in #count_heartbeats inside a namespace Currently the `#count_heartbeat` linter reported the heartbeats until it concluded `error: [declaration] has already been declared` instead of re-elaborating the declaration. --- [Zulip report](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/count_heartbeats.20for.20all.20declarations.20in.20a.20file.3F/near/496303652) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-meta merge-conflict 72/5 Mathlib/Util/CountHeartbeats.lean,MathlibTest/CountHeartbeats.lean 2 17 ['adomani', 'github-actions', 'joneugster', 'leanprover-community-bot-assistant', 'mathlib-bors'] adomani
assignee:adomani
6-38133
6 days ago
6-38134
6 days ago
64-19141
64 days
17715 adomani
author:adomani
feat: the unusedVariableCommand linter This is still work-in-progress, but also help-wanted! The linter reliably flags unused variables: so far, only `example`s fool it (and that is simply because I did not implement a fix, as there are very few `variable`s that are only used in `example`s in mathlib). The work-in-progress part refers to the fact that the linter uses an `IO.Ref` to keep track of variables and this does not work well with editing the file. The linter works on a fresh parse of a file, but becomes out-of-sync with every edit. The help-wanted is to ask for help to make mathlib compliant with the linter, by checking out this branch and PR-ing a few variable removals! [Zulip discussion](https://leanprover.zulipchat.com/#narrow/stream/113488-general/topic/Unused.20variables) --- Known issues: * automatic namespacing and `nonrec` may cause difficulty when the newly introduced declaration is preferred in the term, rather than the original one (see examples here ```bash code -r -g ././././Mathlib/Analysis/SpecialFunctions/Arsinh.lean:183 code -r -g ././././Mathlib/Probability/Independence/Basic.lean:368 ``` where, for instance, `ContinuousOn.arsinh` is used internally instead of `Real.arsinh`). * `mutual` declarations confuse the linter ```bash code -r -g ././././Mathlib/SetTheory/Lists.lean:313 ``` * `code -r -g Mathlib/CategoryTheory/EffectiveEpi/Comp.lean:133:29` * universe annotations confuse the linter: ```bash code -r -g ././././Mathlib/Topology/Category/CompactlyGenerated.lean:53 code -r -g ././././Mathlib/AlgebraicTopology/CechNerve.lean:46 ``` * `inductive`s confusing the linter ```bash code -r -g ././././Mathlib/Deprecated/Subgroup.lean:389 code -r -g ././././Mathlib/FieldTheory/PerfectClosure.lean:55 ``` * `def`s confusing the linter ```bash code -r -g ././././Mathlib/Data/MLList/BestFirst.lean:104 ``` * special typeclass assumptions ```code code -r -g ././././Mathlib/RingTheory/WittVector/Truncated.lean:273 code -r -g ././././Mathlib/Topology/Category/Profinite/Product.lean:79 ``` * not sure what is going on here: ```bash code -r -g ././././Mathlib/RingTheory/WittVector/IsPoly.lean:95 code -r -g ././././Mathlib/Probability/Independence/Basic.lean:368 code -r -g ././././Mathlib/Analysis/Calculus/FDeriv/Star.lean:30 ``` [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-linter merge-conflict 695/22 Mathlib.lean,Mathlib/Algebra/Group/Idempotent.lean,Mathlib/Algebra/GroupWithZero/Idempotent.lean,Mathlib/Data/Finite/Defs.lean,Mathlib/Data/Int/Cast/Field.lean,Mathlib/Geometry/Manifold/IntegralCurve/ExistUnique.lean,Mathlib/Init.lean,Mathlib/MeasureTheory/Function/LpSpace/DomAct/Continuous.lean,Mathlib/NumberTheory/LSeries/PrimesInAP.lean,Mathlib/Order/BoundedOrder/Basic.lean,Mathlib/Order/BoundedOrder/Lattice.lean,Mathlib/Order/BoundedOrder/Monotone.lean,Mathlib/Order/Monotone/Monovary.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter/UnusedVariableCommand.lean,MathlibTest/UnusedVariableCommand.lean,lakefile.lean 17 n/a ['github-actions', 'grunweg', 'leanprover-community-bot-assistant'] nobody
6-16769
6 days ago
unknown
unknown
22909 AntoineChambert-Loir
author:AntoineChambert-Loir
feat(RingTheory/Pure): pure submodules A submodule `N` of an `R`-module is *pure* if all maps `S ⊗[R] N → S ⊗[R] M` deduced by base change from the injection of `N` into `M` are injective, for all `R`-algebras `S`. This is expressed by the class `Submodule.IsPure`. For type theoretic reason, the definition of `Submodule.IsPure` only considers algebras `S` in the same universe as `R`, but `Submodule.IsPure.baseChange_injective` establishes the property for all universes. * `Submodule.IsComplemented.isPure` : a complemented submodule is pure. Co-authored with @mariainesdff --- - [ ] depends on: #22898 - [ ] depends on: #22908 - [x] depends on: #22911 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict blocked-by-other-PR
label:t-algebra$
592/3 Mathlib.lean,Mathlib/Algebra/Algebra/Equiv.lean,Mathlib/RingTheory/Adjoin/FG.lean,Mathlib/RingTheory/Finiteness/Basic.lean,Mathlib/RingTheory/Finiteness/Cardinality.lean,Mathlib/RingTheory/Finiteness/Small.lean,Mathlib/RingTheory/Pure.lean,Mathlib/RingTheory/Spectrum/Prime/RingHom.lean,Mathlib/RingTheory/TensorProduct/Basic.lean,Mathlib/RingTheory/TensorProduct/DirectLimit/FG.lean,Mathlib/RingTheory/TensorProduct/DirectLimit/Small.lean 11 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
6-15600
6 days ago
6-15602
6 days ago
0-1047
17 minutes
23506 Timeroot
author:Timeroot
feat (ModelTheory/Definability): TermDefinable functions Defines `TermDefinable` functions, as functions that can be expressed directly as a term in some interpretation of a language. Shows that this is transitive (as a relationship between structures) and closed under composition of functions. --- Pulled out from #19695. - [x] depends on: #23501 - [ ] depends on: #23502 - [ ] depends on: #23504 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-logic merge-conflict blocked-by-other-PR 191/0 Mathlib/Data/Rel.lean,Mathlib/ModelTheory/Definability.lean,Mathlib/ModelTheory/Semantics.lean,Mathlib/ModelTheory/Syntax.lean,scripts/noshake.json 5 7 ['Timeroot', 'github-actions', 'grunweg', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
6-15377
6 days ago
6-15380
6 days ago
2-32155
2 days
25280 Brian-Nugent
author:Brian-Nugent
feat: add `IsLocalRing.embDim`, the embedding dimension of a local ring This adds the embedding dimension of a local ring and proves basic properties about it. In particular, it proves that if we mod out by an element that is non-zero in the cotangent space, then the embedding dimension drops by exactly one. Co-Authored-By: Jarod Alper [jarod@uw.edu](mailto:jarod@uw.edu) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra merge-conflict
label:t-algebra$
493/2 Mathlib.lean,Mathlib/Algebra/Module/SpanRank.lean,Mathlib/RingTheory/EmbeddingDimension.lean,Mathlib/RingTheory/LocalRing/RingHom/Basic.lean,lake-manifest.json 5 18 ['Brian-Nugent', 'erdOne', 'github-actions', 'leanprover-community-bot-assistant'] nobody
6-13599
6 days ago
8-53929
8 days ago
3-2521
3 days
24105 urkud
author:urkud
feat(Topology/UniformSpace/Path): new file --- - [x] depends on: #24066 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology merge-conflict awaiting-author 117/5 Mathlib.lean,Mathlib/Topology/ContinuousMap/Defs.lean,Mathlib/Topology/Order/ProjIcc.lean,Mathlib/Topology/Path.lean,Mathlib/Topology/UniformSpace/CompactConvergence.lean,Mathlib/Topology/UniformSpace/Path.lean 6 10 ['ADedecker', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'sgouezel', 'urkud'] nobody
6-11152
6 days ago
6-11153
6 days ago
12-77412
12 days
23371 grunweg
author:grunweg
chore: mark `Disjoint.{eq_bot, inter_eq}` simp And add the analogous lemma to `Finset`. Spun out from #22964, hence transitively part of my bordism theory project. Some lemmas there are more conveniently stated with `Disjoint`, which requires tagging at least `inter_eq` with simp. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-order merge-conflict awaiting-author 12/11 Mathlib/Data/Finset/Lattice/Basic.lean,Mathlib/Data/Finset/Lattice/Lemmas.lean,Mathlib/Data/Set/Basic.lean,Mathlib/Data/Set/Disjoint.lean,Mathlib/Order/Disjoint.lean,Mathlib/Topology/Compactification/OnePoint.lean,Mathlib/Topology/Order/OrderClosed.lean 7 31 ['YaelDillies', 'eric-wieser', 'github-actions', 'grunweg', 'j-loreaux', 'leanprover-bot', 'leanprover-community-bot-assistant', 'leanprover-community-mathlib4-bot'] nobody
5-22494
5 days ago
5-22497
5 days ago
32-65400
32 days
24881 smmercuri
author:smmercuri
feat: `InfinitePlace.Extension` API for extensions of infinite places. If `L / K` are fields and `v : InfinitePlace K`, then we define - `v.Extension L` : the subtype of `w : InfinitePlace L` whose restriction to `K` matches `v`. - `isExtension_or_isExtension_conjugate` : if `w` extends `v`, then either `w.embedding` extends `v.embedding` or `conjugate w.embedding` extends `v.embedding` - `IsLift`: class encoding the case where `w` extends `v` and `w.embedding` extends `v.embedding`. - `IsConjugateLift`: class encoding the case where `w` extends `v` and `conjugate w.embedding` extends `v.embedding`. --- - [ ] depends on: #24877 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR 181/0 Mathlib/NumberTheory/NumberField/InfinitePlace/Embeddings.lean,Mathlib/NumberTheory/NumberField/InfinitePlace/Ramification.lean 2 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
5-7757
5 days ago
5-7758
5 days ago
0-1074
17 minutes
24877 smmercuri
author:smmercuri
feat: predicates for extensions of complex embeddings If `L/K`, `ψ : K →+* ℂ`, `φ : L →+* ℂ` we define three predicates asserting ways that `φ` can extend `ψ`. - `IsExtension ψ φ` : the restriction of `φ` to `K` is `ψ`. - `IsMixedExtension ψ φ` : the restriction of `φ` to `K` is `ψ`, `ψ` has real image while `φ` has complex image. - `IsUnmixedExtension ψ φ`: the restriction of `φ` to `K` is `ψ`, `ψ` has real image if and only if `φ` has real image. `IsMixedExtension` and `IsUnmixedExtension` are the `ComplexEmbedding` analogues to ramified and unramified infinite places. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-number-theory merge-conflict 91/0 Mathlib/NumberTheory/NumberField/InfinitePlace/Embeddings.lean 1 7 ['github-actions', 'leanprover-community-bot-assistant', 'smmercuri', 'xroblot'] nobody
5-7757
5 days ago
5-7759
5 days ago
21-40253
21 days
24882 smmercuri
author:smmercuri
feat: `RamifiedExtension` and `UnramifiedExtension` types for `InfinitePlace.Extension`s - `v.RamifiedExtension L` : the subtype of `v.Extension L` consisting of ramified extensions. - `v.UnramifiedExtension L` : the subtype of `v.Extension L` consisting of unramified extensions. --- - [ ] depends on: #24877 - [x] depends on: #24880 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-number-theory merge-conflict blocked-by-other-PR 258/0 Mathlib/NumberTheory/NumberField/InfinitePlace/Embeddings.lean,Mathlib/NumberTheory/NumberField/InfinitePlace/Ramification.lean 2 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
5-7756
5 days ago
5-7757
5 days ago
0-655
10 minutes
25404 grunweg
author:grunweg
perf: benchmarking #24924 Let's see if reverting this shows a similar performance hit. --- Previous summary: [#rss > Benchmark results for mathlib4 @ 💬](https://leanprover.zulipchat.com/#narrow/channel/116290-rss/topic/Benchmark.20results.20for.20mathlib4/near/522168494) Post-merge benchmarking run: https://speed.lean-lang.org/mathlib4/run-detail/772a3867-c7bc-47fe-b380-f5f70e2ccb1b [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) bench-after-CI merge-conflict WIP 26/45 Mathlib/Init.lean,MathlibTest/AssertExists.lean,lakefile.lean,scripts/noshake.json 4 8 ['Vierkantor', 'adomani', 'github-actions', 'grunweg', 'leanprover-bot', 'leanprover-community-bot-assistant', 'leanprover-community-mathlib4-bot', 'mattrobball'] nobody
5-7024
5 days ago
5-7026
5 days ago
0-11
11 seconds
13646 JovanGerb
author:JovanGerb
Lean pr testing 4223 I lowered the instance priorities for `monadError`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict 2/2 lakefile.lean,lean-toolchain 2 2 ['JovanGerb', 'leanprover-bot'] nobody
4-29888
4 days ago
365-77760
1 year ago
0-0
0 seconds
13191 JovanGerb
author:JovanGerb
Lean pr testing 4272 testing more aggressive caching --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor merge-conflict 2/2 lakefile.lean,lean-toolchain 2 19 ['JovanGerb', 'MichaelStollBayreuth', 'leanprover-bot'] nobody
4-29888
4 days ago
380-35792
1 year ago
0-0
0 seconds
13079 JovanGerb
author:JovanGerb
Lean pr testing 4152 Testing some aggressive instance caching. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor merge-conflict 555/723 Mathlib.lean,Mathlib/Algebra/BigOperators/Fin.lean,Mathlib/Algebra/Group/Fin.lean,Mathlib/Algebra/Group/Units/Equiv.lean,Mathlib/Algebra/GroupRingAction/Basic.lean,Mathlib/Algebra/GroupRingAction/Invariant.lean,Mathlib/Algebra/GroupRingAction/Subobjects.lean,Mathlib/Algebra/GroupWithZero/Units/Basic.lean,Mathlib/Algebra/Order/GroupWithZero/WithZero.lean,Mathlib/Algebra/PUnitInstances.lean,Mathlib/Algebra/Polynomial/GroupRingAction.lean,Mathlib/Algebra/Ring/Aut.lean,Mathlib/Algebra/Ring/Subsemiring/Basic.lean,Mathlib/Algebra/Ring/Subsemiring/Pointwise.lean,Mathlib/Analysis/Analytic/Basic.lean,Mathlib/Analysis/Calculus/FDeriv/Mul.lean,Mathlib/CategoryTheory/ComposableArrows.lean,Mathlib/Combinatorics/Enumerative/Composition.lean,Mathlib/Combinatorics/SetFamily/HarrisKleitman.lean,Mathlib/Combinatorics/SetFamily/Intersecting.lean,Mathlib/Combinatorics/SimpleGraph/Clique.lean,Mathlib/Computability/RegularExpressions.lean,Mathlib/Control/Random.lean,Mathlib/Data/Fin/Basic.lean,Mathlib/Data/Fin/FlagRange.lean,Mathlib/Data/Fin/OrderHom.lean,Mathlib/Data/Fin/SuccPred.lean,Mathlib/Data/Fin/Tuple/Basic.lean,Mathlib/Data/Fin/VecNotation.lean,Mathlib/Data/Finset/Sort.lean,Mathlib/Data/Finsupp/Fin.lean,Mathlib/Data/Fintype/Basic.lean,Mathlib/Data/Fintype/Card.lean,Mathlib/Data/Fintype/Fin.lean,Mathlib/Data/Fintype/Units.lean,Mathlib/Data/List/Cycle.lean,Mathlib/Data/List/Indexes.lean,Mathlib/Data/List/NodupEquivFin.lean,Mathlib/Data/List/OfFn.lean,Mathlib/Data/Nat/Bits.lean,Mathlib/Data/Nat/Bitwise.lean,Mathlib/Data/ZMod/Basic.lean,Mathlib/FieldTheory/Fixed.lean,Mathlib/GroupTheory/FreeGroup/Basic.lean,Mathlib/GroupTheory/GroupAction/ConjAct.lean,Mathlib/GroupTheory/GroupAction/Hom.lean,Mathlib/GroupTheory/OrderOfElement.lean,Mathlib/GroupTheory/Perm/Fin.lean,Mathlib/GroupTheory/Perm/List.lean,Mathlib/GroupTheory/Perm/Support.lean,Mathlib/LinearAlgebra/Dimension/Free.lean,Mathlib/LinearAlgebra/FreeModule/PID.lean,Mathlib/LinearAlgebra/TensorAlgebra/ToTensorPower.lean,Mathlib/LinearAlgebra/TensorPower.lean,Mathlib/Logic/Equiv/Fin.lean,Mathlib/ModelTheory/Semantics.lean,Mathlib/Order/Fin.lean,Mathlib/Order/Grade.lean,Mathlib/Order/JordanHolder.lean,Mathlib/Order/RelSeries.lean,Mathlib/Order/SuccPred/LinearLocallyFinite.lean,Mathlib/Order/SupIndep.lean,Mathlib/RingTheory/Congruence.lean,Mathlib/RingTheory/DedekindDomain/AdicValuation.lean,Mathlib/Tactic/Says.lean,Mathlib/Topology/UniformSpace/CompactConvergence.lean,Shake/Main.lean,lakefile.lean,lean-toolchain,test/CompileInductive.lean 70 4 ['JovanGerb', 'leanprover-bot'] nobody
4-29888
4 days ago
381-35556
1 year ago
0-0
0 seconds
22529 kmill
author:kmill
Lean pr testing 7313 (for benchmarking) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict 32/16 Mathlib/Algebra/Field/Subfield/Defs.lean,Mathlib/Algebra/Ring/Equiv.lean,Mathlib/CategoryTheory/Presentable/Basic.lean,Mathlib/CategoryTheory/Triangulated/Adjunction.lean,Mathlib/FieldTheory/IsAlgClosed/Basic.lean,Mathlib/FieldTheory/IsSepClosed.lean,Mathlib/Order/Hom/Bounded.lean,Mathlib/RingTheory/NonUnitalSubring/Defs.lean,Mathlib/RingTheory/RingInvo.lean,lake-manifest.json,lakefile.lean,lean-toolchain 12 3 ['github-actions', 'kmill', 'leanprover-bot'] nobody
4-29888
4 days ago
97-57167
3 months ago
0-0
0 seconds
22177 JovanGerb
author:JovanGerb
Lean pr testing 7181 Testing the effect of abstracting proofs in theorem statements --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict 425/60 Mathlib/AlgebraicGeometry/FunctionField.lean,Mathlib/AlgebraicGeometry/Morphisms/AffineAnd.lean,Mathlib/CategoryTheory/SmallObject/Iteration/Nonempty.lean,Mathlib/FieldTheory/Galois/Profinite.lean,Mathlib/FieldTheory/IntermediateField/Adjoin/Basic.lean,Mathlib/FieldTheory/Laurent.lean,Mathlib/FieldTheory/SplittingField/Construction.lean,Mathlib/FieldTheory/SplittingField/IsSplittingField.lean,Mathlib/GroupTheory/Perm/Cycle/Basic.lean,Mathlib/LinearAlgebra/LinearPMap.lean,Mathlib/MeasureTheory/Function/ConditionalExpectation/AEMeasurable.lean,Mathlib/MeasureTheory/Function/ConditionalExpectation/CondexpL1.lean,Mathlib/MeasureTheory/Function/ConditionalExpectation/CondexpL2.lean,Mathlib/RingTheory/Adjoin/Tower.lean,Mathlib/RingTheory/HahnSeries/Summable.lean,lake-manifest.json,lakefile.lean,lean-toolchain 18 3 ['JovanGerb', 'github-actions', 'leanprover-bot'] nobody
4-29888
4 days ago
107-76302
3 months ago
0-0
0 seconds
15598 kmill
author:kmill
Lean pr testing 4938 Creating a PR for benchmarking --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict 6/8 Counterexamples/ZeroDivisorsInAddMonoidAlgebras.lean,Mathlib/AlgebraicTopology/DoldKan/Degeneracies.lean,Mathlib/MeasureTheory/Order/UpperLower.lean,Mathlib/NumberTheory/WellApproximable.lean,lake-manifest.json,lakefile.lean,lean-toolchain 7 2 ['kmill', 'leanprover-bot'] nobody
4-29888
4 days ago
306-3670
10 months ago
0-0
0 seconds
23129 JovanGerb
author:JovanGerb
Lean pr testing 7585 Some optimization in `simp` proof term generation. I found this by looking at `map_comp_cotangentComplex_baseChange` in `JacobiZariski.lean` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict 15/14 Mathlib/Condensed/Discrete/Colimit.lean,Mathlib/RingTheory/DedekindDomain/SelmerGroup.lean,lake-manifest.json,lakefile.lean,lean-toolchain 5 4 ['github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot'] nobody
4-29888
4 days ago
80-6602
2 months ago
0-0
0 seconds
23203 Kha
author:Kha
leanprover/lean4#7597 benchmarking ignore me merge-conflict 4/4 lake-manifest.json,lakefile.lean,lean-toolchain 3 3 ['Kha', 'github-actions', 'leanprover-bot'] nobody
4-29888
4 days ago
80-6066
2 months ago
0-0
0 seconds
23644 JovanGerb
author:JovanGerb
Lean pr testing 7804 Testing an optimization in `simp` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict 4/4 lake-manifest.json,lakefile.lean,lean-toolchain 3 3 ['github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot'] nobody
4-29888
4 days ago
66-75572
2 months ago
0-2933
48 minutes
24128 kmill
author:kmill
Lean pr testing 7991 (for benchmarking) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict 28/85 Counterexamples/CliffordAlgebraNotInjective.lean,Mathlib/Algebra/Algebra/NonUnitalSubalgebra.lean,Mathlib/Algebra/Algebra/Subalgebra/Directed.lean,Mathlib/Algebra/Free.lean,Mathlib/Algebra/Homology/HomotopyCategory/HomComplexShift.lean,Mathlib/Algebra/Module/DedekindDomain.lean,Mathlib/Algebra/Order/AddGroupWithTop.lean,Mathlib/Algebra/Order/Group/Int/Sum.lean,Mathlib/Algebra/RingQuot.lean,Mathlib/Algebra/Star/NonUnitalSubalgebra.lean,Mathlib/AlgebraicGeometry/Morphisms/QuasiCompact.lean,Mathlib/AlgebraicTopology/FundamentalGroupoid/Basic.lean,Mathlib/Analysis/Analytic/CPolynomialDef.lean,Mathlib/Analysis/BoxIntegral/Partition/Additive.lean,Mathlib/Analysis/CStarAlgebra/PositiveLinearMap.lean,Mathlib/Analysis/Convex/Combination.lean,Mathlib/Analysis/InnerProductSpace/Projection.lean,Mathlib/Analysis/SpecialFunctions/Gamma/Beta.lean,Mathlib/Analysis/SpecificLimits/Normed.lean,Mathlib/CategoryTheory/ComposableArrows.lean,Mathlib/CategoryTheory/EqToHom.lean,Mathlib/CategoryTheory/Localization/CalculusOfFractions.lean,Mathlib/CategoryTheory/Quotient/Linear.lean,Mathlib/CategoryTheory/Sites/Plus.lean,Mathlib/CategoryTheory/Subobject/Basic.lean,Mathlib/CategoryTheory/Subobject/Lattice.lean,Mathlib/CategoryTheory/Triangulated/Opposite/Basic.lean,Mathlib/CategoryTheory/Triangulated/Opposite/Functor.lean,Mathlib/Combinatorics/Additive/CauchyDavenport.lean,Mathlib/Combinatorics/Enumerative/IncidenceAlgebra.lean,Mathlib/Combinatorics/Quiver/Push.lean,Mathlib/Combinatorics/SimpleGraph/ConcreteColorings.lean,Mathlib/Computability/TuringMachine.lean,Mathlib/Data/Fintype/CardEmbedding.lean,Mathlib/Data/Fintype/List.lean,Mathlib/Data/Int/Bitwise.lean,Mathlib/Data/List/NodupEquivFin.lean,Mathlib/Data/QPF/Multivariate/Constructions/Cofix.lean,Mathlib/Data/QPF/Univariate/Basic.lean,Mathlib/Geometry/Euclidean/Basic.lean,Mathlib/GroupTheory/CoprodI.lean,Mathlib/GroupTheory/Coset/Basic.lean,Mathlib/GroupTheory/GroupAction/Quotient.lean,Mathlib/GroupTheory/MonoidLocalization/Order.lean,Mathlib/GroupTheory/OrderOfElement.lean,Mathlib/GroupTheory/OreLocalization/Basic.lean,Mathlib/LinearAlgebra/BilinearMap.lean,Mathlib/LinearAlgebra/LinearIndependent/Defs.lean,Mathlib/MeasureTheory/VectorMeasure/Basic.lean,Mathlib/ModelTheory/DirectLimit.lean,Mathlib/ModelTheory/Encoding.lean,Mathlib/NumberTheory/LucasLehmer.lean,Mathlib/Order/SuccPred/Archimedean.lean,Mathlib/Probability/Independence/Basic.lean,Mathlib/Probability/Moments/ComplexMGF.lean,Mathlib/Probability/ProbabilityMassFunction/Binomial.lean,Mathlib/RingTheory/AlgebraicIndependent/TranscendenceBasis.lean,Mathlib/RingTheory/Filtration.lean,Mathlib/RingTheory/FractionalIdeal/Norm.lean,Mathlib/RingTheory/OreLocalization/Basic.lean,Mathlib/RingTheory/Polynomial/UniqueFactorization.lean,Mathlib/RingTheory/WittVector/FrobeniusFractionField.lean,Mathlib/Topology/Algebra/InfiniteSum/Module.lean,Mathlib/Topology/Germ.lean,lean-toolchain 65 11 ['github-actions', 'kmill', 'leanprover-bot', 'leanprover-community-bot-assistant'] nobody
4-29888
4 days ago
50-35519
1 month ago
0-0
0 seconds
25352 kmill
author:kmill
Lean pr testing 8373 (for benchmarking) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict 16/14 Mathlib/CategoryTheory/Monad/Comonadicity.lean,Mathlib/CategoryTheory/Monad/Monadicity.lean,Mathlib/Data/PFunctor/Univariate/M.lean,Mathlib/FieldTheory/Finite/GaloisField.lean,Mathlib/GroupTheory/MonoidLocalization/Basic.lean,Mathlib/LinearAlgebra/FiniteDimensional/Basic.lean,Mathlib/MeasureTheory/VectorMeasure/Decomposition/Jordan.lean,Mathlib/RingTheory/Extension/Presentation/Basic.lean,Mathlib/Tactic/ModCases.lean,lake-manifest.json,lakefile.lean,lean-toolchain 12 6 ['github-actions', 'kmill', 'leanprover-bot', 'leanprover-community-bot-assistant'] nobody
4-29888
4 days ago
7-59000
7 days ago
0-0
0 seconds
16062 adomani
author:adomani
Test/ci olean size Tests for oleans --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) CI merge-conflict awaiting-author WIP 114/0 .github/build.in.yml,.github/workflows/bors.yml,.github/workflows/build.yml,.github/workflows/build_fork.yml,scripts/olean_comparison.sh 5 4 ['Parcly-Taxel', 'adomani', 'github-actions', 'leanprover-community-bot-assistant'] nobody
3-59392
3 days ago
3-59393
3 days ago
0-16
16 seconds
16020 adomani
author:adomani
feat: compare PR `olean`s size with `master` Adds two CI steps: * `print the sizes of the oleans` that prints the sizes of all the folders containing `Mathlib` `.olean`s; * `compare oleans` that compares the sizes of the previous step with the corresponding sizes on `master`. In the test runs, the two steps have taken at most 3 seconds combined (the first is virtually instantaneous, the second one depends on `curl` to find a job id and on `gh` to retrieve the logs of a previous CI run -- everything else appears to be negligible). This hopefully helps finding out if some PR is bloating up the `.olean`s. See [this Zulip discussion](https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/Error.3A.20No.20space.20left.20on.20device/near/463792355) for a PR of mine that prompted this check. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) CI merge-conflict 120/0 .github/build.in.yml,.github/workflows/bors.yml,.github/workflows/build.yml,.github/workflows/build_fork.yml,scripts/olean_comparison.sh 5 50 ['Vtec234', 'YaelDillies', 'adomani', 'bryangingechen', 'github-actions', 'grunweg', 'kim-em', 'leanprover-community-bot-assistant', 'mattrobball'] nobody
3-59392
3 days ago
3-59394
3 days ago
285-26861
285 days
19633 grunweg
author:grunweg
fix(CI): build the Archive and Counterexamples with --wfail also This appears to be an oversight --- which has no consequences right now (the check for noisy output later would catch any warnings), but fixing it doesn't hurt either. [Zulip discussion](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/No.20.60--wfail.60.20when.20building.20archive). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) CI awaiting-CI easy merge-conflict delegated 20/8 .github/build.in.yml,.github/workflows/bors.yml,.github/workflows/build.yml,.github/workflows/build_fork.yml 4 6 ['adomani', 'github-actions', 'grunweg', 'kim-em', 'leanprover-community-bot-assistant', 'mathlib-bors'] nobody
3-59146
3 days ago
3-59148
3 days ago
7-42070
7 days
25507 eric-wieser
author:eric-wieser
chore(RingTheory/Valuation): golf using `Con` This has no particular motivation besides seeing if `Con` is a performant substitute. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) bench-after-CI t-algebra merge-conflict
label:t-algebra$
20/35 Mathlib/RingTheory/Valuation/ValuationRing.lean 1 2 ['github-actions', 'leanprover-community-bot-assistant'] nobody
3-50871
3 days ago
3-50872
3 days ago
0-0
0 seconds
7596 alreadydone
author:alreadydone
feat: covering maps from properly discontinuous actions and discrete subgroups --- - [x] depends on: #23236 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) file-removed t-topology merge-conflict 351/21 Mathlib.lean,Mathlib/Analysis/SpecialFunctions/Complex/Circle.lean,Mathlib/Topology/Algebra/ConstMulAction.lean,Mathlib/Topology/Algebra/Group/Pointwise.lean,Mathlib/Topology/Covering/AddCircle.lean,Mathlib/Topology/Covering/Basic.lean,Mathlib/Topology/Covering/Galois.lean,Mathlib/Topology/Homotopy/Lifting.lean,Mathlib/Topology/Instances/AddCircle.lean 9 17 ['ADedecker', 'alreadydone', 'digama0', 'github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'tb65536'] nobody
3-27315
3 days ago
3-27317
3 days ago
48-80629
48 days
25432 riccardobrasca
author:riccardobrasca
Rb cyclo --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict WIP 1320/2 Mathlib.lean,Mathlib/Algebra/Module/Equiv/Defs.lean,Mathlib/Data/ZMod/QuotientRing.lean,Mathlib/GroupTheory/Exponent.lean,Mathlib/LinearAlgebra/Dimension/Finrank.lean,Mathlib/NumberTheory/NumberField/Ideal/KummerDedekind.lean,Mathlib/NumberTheory/RamificationInertia/Basic.lean,Mathlib/Order/Atoms.lean,Mathlib/RingTheory/AdjoinRoot.lean,Mathlib/RingTheory/DedekindDomain/Ideal.lean,Mathlib/RingTheory/Ideal/Int.lean,Mathlib/RingTheory/Ideal/Over.lean,Mathlib/RingTheory/Ideal/Span.lean,Mathlib/Stuff/Cyclotomic.lean,Mathlib/Stuff/Eleven.lean,Mathlib/Stuff/Factorization.lean,Mathlib/Stuff/Inertia.lean,Mathlib/Stuff/Minkowski.lean,Mathlib/Stuff/OrderOf.lean,Mathlib/Stuff/Seven.lean,Mathlib/Stuff/Thirteen.lean 21 3 ['github-actions', 'leanprover-community-bot-assistant'] nobody
3-8828
3 days ago
3-8830
3 days ago
0-0
0 seconds
12799 jstoobysmith
author:jstoobysmith
feat(LinearAlgebra/UnitaryGroup): Add properties of Special Unitary Group Add properties of the special unitary group, mirroring the properties of found in Algebra/Star/Unitary.lean. In particular, I add an instance of `specialUnitaryGroup` as a `Group`, `Star`, `InvolutiveStar`, and `StarMul`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-algebra merge-conflict please-adopt awaiting-author
label:t-algebra$
78/0 Mathlib/LinearAlgebra/UnitaryGroup.lean 1 8 ['chrisflav', 'jcommelin', 'leanprover-community-bot-assistant'] nobody
2-67738
2 days ago
2-67740
2 days ago
9-22007
9 days
23961 FR-vdash-bot
author:FR-vdash-bot
refactor: unbundle algebra from `ENormed*` Further speed up the search in the algebraic typeclass hierarchy by avoiding searching for `TopologicalSpace`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) slow-typeclass-synthesis maintainer-merge t-algebra t-analysis merge-conflict awaiting-author
label:t-algebra$
32/25 Mathlib/Analysis/CStarAlgebra/CStarMatrix.lean,Mathlib/Analysis/Normed/Group/Basic.lean,Mathlib/Analysis/Normed/Group/Continuity.lean,Mathlib/Analysis/NormedSpace/IndicatorFunction.lean,Mathlib/MeasureTheory/Function/LpSeminorm/Basic.lean 5 12 ['FR-vdash-bot', 'github-actions', 'grunweg', 'jcommelin', 'leanprover-bot', 'leanprover-community-bot-assistant'] nobody
2-46984
2 days ago
2-46984
2 days ago
17-72244
17 days
23709 plp127
author:plp127
feat: `Nat.findFrom` This PR adds `Nat.findFrom`, which is like `Nat.find`, but starting from an arbitrary `k` instead of `0`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-data merge-conflict 190/47 Mathlib/Data/Nat/Find.lean 1 2 ['github-actions', 'leanprover-community-bot-assistant'] nobody
2-33027
2 days ago
2-33029
2 days ago
62-25661
62 days
25038 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. --- - [x] depends on: #25080 - [x] depends on: #25149 - [x] depends on: #25316 - [x] depends on: #25388 - [ ] depends on: #25527 - [x] depends on: #25528 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-number-theory merge-conflict blocked-by-other-PR WIP 406/1 Mathlib.lean,Mathlib/Data/ZMod/QuotientRing.lean,Mathlib/GroupTheory/Exponent.lean,Mathlib/LinearAlgebra/Dimension/Finrank.lean,Mathlib/NumberTheory/NumberField/Ideal/KummerDedekind.lean,Mathlib/NumberTheory/RamificationInertia/Basic.lean,Mathlib/Order/Atoms.lean,Mathlib/RingTheory/AdjoinRoot.lean,Mathlib/RingTheory/DedekindDomain/Ideal.lean,Mathlib/RingTheory/Ideal/Int.lean,Mathlib/RingTheory/Ideal/Over.lean,Mathlib/RingTheory/Ideal/Span.lean 12 6 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] riccardobrasca
assignee:riccardobrasca
2-32260
2 days ago
3-8955
3 days ago
0-9855
2 hours
25340 dupuisf
author:dupuisf
chore(Analysis/Convex): move files pertaining to convex/concave functions to their own folder This PR creates a new folder under `Analysis/Convex` called `Analysis/Convex/Function`, which includes files that are mostly or entirely about convex/concave functions (as opposed to convex sets). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-convex-geometry merge-conflict 4264/4155 Mathlib.lean,Mathlib/Analysis/Convex/Continuous.lean,Mathlib/Analysis/Convex/Deriv.lean,Mathlib/Analysis/Convex/Exposed.lean,Mathlib/Analysis/Convex/Extrema.lean,Mathlib/Analysis/Convex/Function.lean,Mathlib/Analysis/Convex/Function/Basic.lean,Mathlib/Analysis/Convex/Function/Continuous.lean,Mathlib/Analysis/Convex/Function/Deriv.lean,Mathlib/Analysis/Convex/Function/Extrema.lean,Mathlib/Analysis/Convex/Function/Integral.lean,Mathlib/Analysis/Convex/Function/Jensen.lean,Mathlib/Analysis/Convex/Function/Mul.lean,Mathlib/Analysis/Convex/Function/Piecewise.lean,Mathlib/Analysis/Convex/Function/Quasiconvex.lean,Mathlib/Analysis/Convex/Function/Slope.lean,Mathlib/Analysis/Convex/Function/Strong.lean,Mathlib/Analysis/Convex/Integral.lean,Mathlib/Analysis/Convex/Jensen.lean,Mathlib/Analysis/Convex/Mul.lean,Mathlib/Analysis/Convex/Piecewise.lean,Mathlib/Analysis/Convex/Quasiconvex.lean,Mathlib/Analysis/Convex/Slope.lean,Mathlib/Analysis/Convex/SpecificFunctions/Basic.lean,Mathlib/Analysis/Convex/SpecificFunctions/Deriv.lean,Mathlib/Analysis/Convex/Strong.lean,Mathlib/Analysis/MeanInequalities.lean,Mathlib/Analysis/MeanInequalitiesPow.lean,Mathlib/Analysis/Normed/Module/Convex.lean,Mathlib/Analysis/Seminorm.lean,Mathlib/Analysis/SpecialFunctions/Log/NegMulLog.lean,Mathlib/Analysis/SpecialFunctions/Pochhammer.lean,Mathlib/MeasureTheory/Measure/Decomposition/IntegralRNDeriv.lean,Mathlib/NumberTheory/Harmonic/GammaDeriv.lean 34 2 ['github-actions', 'leanprover-community-bot-assistant'] nobody
2-32212
2 days ago
2-32214
2 days ago
6-40169
6 days
24808 JovanGerb
author:JovanGerb
lean pr testing 8294 Testing a cache optimization in `isDefEq`, to avoid exponential blowup during unification. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict 243/98 Mathlib.lean,Mathlib/Algebra/BigOperators/Group/Finset/Basic.lean,Mathlib/Algebra/BigOperators/Group/Finset/Preimage.lean,Mathlib/Algebra/BigOperators/Intervals.lean,Mathlib/Algebra/Group/Submonoid/Basic.lean,Mathlib/Algebra/GroupWithZero/Basic.lean,Mathlib/Algebra/GroupWithZero/Defs.lean,Mathlib/Algebra/GroupWithZero/NeZero.lean,Mathlib/Algebra/Homology/DifferentialObject.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Affine/Formula.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Affine/Point.lean,Mathlib/Analysis/Complex/ValueDistribution/CharacteristicFunction.lean,Mathlib/Analysis/InnerProductSpace/Spectrum.lean,Mathlib/Analysis/LConvolution.lean,Mathlib/Analysis/NormedSpace/Alternating/Curry.lean,Mathlib/CategoryTheory/Limits/VanKampen.lean,Mathlib/Data/Finset/Fold.lean,Mathlib/Data/Finset/Image.lean,Mathlib/Data/Int/Init.lean,Mathlib/Data/Matrix/Mul.lean,Mathlib/Data/Nat/Factorization/Basic.lean,Mathlib/Data/Set/Function.lean,Mathlib/Data/Set/Image.lean,Mathlib/Data/Vector/MapLemmas.lean,Mathlib/Data/ZMod/Basic.lean,Mathlib/MeasureTheory/Group/Convolution.lean,Mathlib/MeasureTheory/Group/IntegralConvolution.lean,Mathlib/NumberTheory/ArithmeticFunction.lean,Mathlib/NumberTheory/Divisors.lean,Mathlib/Probability/Distributions/Gaussian/Real.lean,Mathlib/Topology/Algebra/InfiniteSum/NatInt.lean,Shake/Main.lean,lake-manifest.json,lakefile.lean,lean-toolchain 35 21 ['JovanGerb', 'adomani', 'github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot'] nobody
2-686
2 days ago
2-686
2 days ago
0-11360
3 hours
13994 grunweg
author:grunweg
chore(Topology): replace continuity -> fun_prop Addresses a few porting notes; I expect also a substantial speed-up of some proofs. Change a few default values of proof fields from `continuity` to `fun_prop`; this required a few fix-ups downstream. (I checked a few instances; the failure seems related to `Continuous.subtype_mk` not always firing.) This is almost (but not fully) exhaustive. ---------- One proof gets partially un-automated (cont. -> partial fun_prop); if desired, I can revert this change. - [x] depends on: #11092 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-topology merge-conflict 105/20 Mathlib/Analysis/Distribution/FourierSchwartz.lean,Mathlib/Analysis/Matrix.lean,Mathlib/Dynamics/Flow.lean,Mathlib/Geometry/RingedSpace/OpenImmersion.lean,Mathlib/Topology/Algebra/Field.lean,Mathlib/Topology/Algebra/Monoid.lean,Mathlib/Topology/Category/TopCat/Limits/Basic.lean,Mathlib/Topology/Category/TopCat/Limits/Pullbacks.lean,Mathlib/Topology/ContinuousMap/Basic.lean,Mathlib/Topology/ContinuousMap/Bounded/Basic.lean,Mathlib/Topology/ContinuousMap/Compact.lean,Mathlib/Topology/ContinuousMap/StoneWeierstrass.lean,Mathlib/Topology/ExtremallyDisconnected.lean,Mathlib/Topology/Homotopy/HomotopyGroup.lean,Mathlib/Topology/Homotopy/Path.lean,Mathlib/Topology/Instances/RealVectorSpace.lean,Mathlib/Topology/MetricSpace/Perfect.lean,Mathlib/Topology/UnitInterval.lean 18 12 ['MichaelStollBayreuth', 'github-actions', 'grunweg', 'j-loreaux', 'leanprover-bot', 'leanprover-community-mathlib4-bot', 'urkud'] nobody
1-50885
1 day ago
276-70516
9 months ago
28-21477
28 days
21734 adomani
author:adomani
fix(PR summary): checkout GITHUB_SHA This should make the version of the script that is used on PRs more stable. Suggested by Eric Wieser on [Zulip](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/messageFile.2Emd/near/498941855). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) CI merge-conflict awaiting-author WIP 2/1 .github/workflows/PR_summary.yml 1 2 ['github-actions', 'leanprover-community-bot-assistant'] nobody
1-48879
1 day ago
1-48881
1 day ago
0-6023
1 hour
25012 urkud
author:urkud
refactor(*): migrate from `Matrix.toLin'` to `Matrix.mulVecLin` or `Matrix.mulVec` whenever we don't need the `LinearEquiv.symm` part. See [Zulip discussion](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/Matrix.2EtoLin'.20vs.20Matrix.2EmulVecLin/with/515188548). It makes sense to have only one normal form, and `Matrix.toLin'` has an extra `DecidableEq` assumption. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict 154/122 Mathlib/Algebra/Lie/Matrix.lean,Mathlib/Algebra/Module/Equiv/Basic.lean,Mathlib/Analysis/CStarAlgebra/Matrix.lean,Mathlib/Analysis/Matrix.lean,Mathlib/Combinatorics/SimpleGraph/LapMatrix.lean,Mathlib/Data/Matrix/Rank.lean,Mathlib/LinearAlgebra/Basis/Defs.lean,Mathlib/LinearAlgebra/Determinant.lean,Mathlib/LinearAlgebra/Finsupp/VectorSpace.lean,Mathlib/LinearAlgebra/FreeModule/Finite/Matrix.lean,Mathlib/LinearAlgebra/Matrix/BilinearForm.lean,Mathlib/LinearAlgebra/Matrix/Charpoly/Minpoly.lean,Mathlib/LinearAlgebra/Matrix/Diagonal.lean,Mathlib/LinearAlgebra/Matrix/Gershgorin.lean,Mathlib/LinearAlgebra/Matrix/SesquilinearForm.lean,Mathlib/LinearAlgebra/Matrix/SpecialLinearGroup.lean,Mathlib/LinearAlgebra/Matrix/ToLin.lean,Mathlib/LinearAlgebra/Matrix/ToLinearEquiv.lean,Mathlib/LinearAlgebra/UnitaryGroup.lean,Mathlib/MeasureTheory/Measure/Lebesgue/Basic.lean,Mathlib/RingTheory/Smooth/StandardSmooth.lean 21 3 ['github-actions', 'leanprover-community-bot-assistant'] nobody
1-27046
1 day ago
1-27048
1 day ago
15-74981
15 days
24434 joelriou
author:joelriou
feat(CategoryTheory): effectiveness of descent Co-authored-by: Christian Merten [christian@merten.dev](mailto:christian@merten.dev) --- - [ ] depends on: #24411 - [ ] depends on: #24382 - [ ] depends on: #24384 - [ ] depends on: #13539 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-category-theory merge-conflict blocked-by-other-PR WIP 4052/66 Mathlib.lean,Mathlib/CategoryTheory/Bicategory/Adjunction/Adj.lean,Mathlib/CategoryTheory/Bicategory/Adjunction/BaseChange.lean,Mathlib/CategoryTheory/Bicategory/Adjunction/Basic.lean,Mathlib/CategoryTheory/Bicategory/Adjunction/Mate.lean,Mathlib/CategoryTheory/Bicategory/Functor/Cat.lean,Mathlib/CategoryTheory/Bicategory/Functor/LocallyDiscrete.lean,Mathlib/CategoryTheory/Bicategory/Functor/Strict.lean,Mathlib/CategoryTheory/Bicategory/Opposite.lean,Mathlib/CategoryTheory/CommSq.lean,Mathlib/CategoryTheory/Limits/Shapes/Pullback/CommSq.lean,Mathlib/CategoryTheory/Sites/Descent/DescentData.lean,Mathlib/CategoryTheory/Sites/Descent/DescentDataAsCoalgebra.lean,Mathlib/CategoryTheory/Sites/Descent/DescentDataDoublePrime.lean,Mathlib/CategoryTheory/Sites/Descent/DescentDataPrime.lean,Mathlib/CategoryTheory/Sites/Descent/IsPrestack.lean,Mathlib/CategoryTheory/Sites/Descent/IsStack.lean,Mathlib/CategoryTheory/Sites/Descent/ModuleCat.lean,Mathlib/CategoryTheory/Sites/Descent/PullbackStruct.lean 19 8 ['callesonne', 'github-actions', 'joelriou', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
1-21667
1 day ago
2-32904
2 days ago
0-0
0 seconds
16303 grunweg
author:grunweg
feat(CI): check for badly formatted titles or missing/contradictory labels --- The zulip workflow is entirely cargo-culted from #16296; please review carefully. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) CI merge-conflict awaiting-author 325/0 .github/build.in.yml,Mathlib.lean,Mathlib/Tactic.lean,Mathlib/Tactic/Linter/ValidatePRTitle.lean,MathlibTest/ValidatePRTitle.lean,lakefile.lean,scripts/README.md,scripts/check-title-labels.lean 8 44 ['Command-Master', 'adomani', 'bryangingechen', 'edegeltje', 'github-actions', 'grunweg', 'joneugster', 'leanprover-community-bot-assistant'] bryangingechen
assignee:bryangingechen
0-54766
15 hours ago
0-54767
15 hours ago
78-54824
78 days
14752 AntoineChambert-Loir
author:AntoineChambert-Loir
fix(Topology/Algebra/Valued): repair definition of Valued Following a [discussion on Zulip](https://leanprover.zulipchat.com/#narrow/stream/116395-maths/topic/Question.20about.20.60Valued.2Eis_topological_valuation.60), we modify the definition of the field `is_topological_valuation` of `Valued` insisting that the element $\gamma$ showing up there is in the subgroup generated by the image of the valuation map. Co-authored-by: @faenuccio - [ ] depends on: #25496 t-algebra t-topology merge-conflict blocked-by-other-PR WIP
label:t-algebra$
1166/301 Mathlib.lean,Mathlib/Algebra/GroupWithZero/Range.lean,Mathlib/NumberTheory/NumberField/FinitePlaces.lean,Mathlib/RingTheory/LaurentSeries.lean,Mathlib/RingTheory/Valuation/Basic.lean,Mathlib/RingTheory/Valuation/RankOne.lean,Mathlib/Topology/Algebra/Valued/LocallyCompact.lean,Mathlib/Topology/Algebra/Valued/NormedValued.lean,Mathlib/Topology/Algebra/Valued/ValuationTopology.lean,Mathlib/Topology/Algebra/Valued/ValuedField.lean,Mathlib/Topology/UniformSpace/AbstractCompletion.lean,docs/references.bib 12 28 ['AntoineChambert-Loir', 'faenuccio', 'github-actions', 'jcommelin', 'kbuzzard', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot', 'riccardobrasca'] riccardobrasca
assignee:riccardobrasca
0-53401
14 hours ago
0-53403
14 hours ago
1-33784
1 day
23394 BoltonBailey
author:BoltonBailey
chore(Data/Int/WithZero): fix erw --- Removing an `erw`. This is my first time doing this, so please tell me if I am doing something wrong here (e.g. should the new lemma be `simp`?). [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) tech debt merge-conflict 5/4 Mathlib/Algebra/Group/WithOne/Defs.lean,Mathlib/Algebra/GroupWithZero/WithZero.lean,Mathlib/Data/Int/WithZero.lean 3 19 ['BoltonBailey', 'Ruben-VandeVelde', 'eric-wieser', 'fpvandoorn', 'github-actions', 'grunweg', 'leanprover-community-bot-assistant'] nobody
0-50895
14 hours ago
0-50897
14 hours ago
52-38111
52 days
22656 101damnations
author:101damnations
feat(RepresentationTheory/Homological/GroupHomology/Functoriality): the degree 1 part of the corestriction-coinflation exact sequence Given a `G`-representation `A` and a normal subgroup `S` of `G`, this PR defines the corestriction-coinflation short complex `H₁(S, A) ⟶ H₁(G, A) ⟶ H₁(G ⧸ S, A_S)` induced by the natural inclusion `S → G` and projections `G → G / S, A → A_S`. We proves it's exact, and that the righthand map is an epimorphism. --- - [ ] depends on: #22651 - [ ] depends on: #22652 - [ ] depends on: #22654 - [x] depends on: #21732 - [ ] depends on: #21733 - [ ] depends on: #21735 - [ ] depends on: #21736 - [ ] depends on: #21738 - [ ] depends on: #21740 - [ ] depends on: #21752 - [ ] depends on: #21754 - [ ] depends on: #21755 - [ ] depends on: #21757 - [ ] depends on: #21759 - [ ] depends on: #21763 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-algebra merge-conflict blocked-by-other-PR
label:t-algebra$
3593/965 Mathlib.lean,Mathlib/Algebra/BigOperators/Fin.lean,Mathlib/Algebra/Homology/ShortComplex/ModuleCat.lean,Mathlib/CategoryTheory/Action/Basic.lean,Mathlib/CategoryTheory/Action/Concrete.lean,Mathlib/CategoryTheory/Action/Monoidal.lean,Mathlib/CategoryTheory/Monoidal/Types/Basic.lean,Mathlib/Data/Finsupp/Basic.lean,Mathlib/GroupTheory/QuotientGroup/Defs.lean,Mathlib/LinearAlgebra/Finsupp/Defs.lean,Mathlib/RepresentationTheory/Basic.lean,Mathlib/RepresentationTheory/Coinvariants.lean,Mathlib/RepresentationTheory/GroupCohomology/Basic.lean,Mathlib/RepresentationTheory/GroupCohomology/Resolution.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/Basic.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/Functoriality.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/Hilbert90.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/LowDegree.lean,Mathlib/RepresentationTheory/Homological/GroupHomology/Basic.lean,Mathlib/RepresentationTheory/Homological/GroupHomology/Functoriality.lean,Mathlib/RepresentationTheory/Homological/GroupHomology/LowDegree.lean,Mathlib/RepresentationTheory/Homological/Resolution.lean,Mathlib/RepresentationTheory/Invariants.lean,Mathlib/RepresentationTheory/Rep.lean 24 n/a ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
0-41043
11 hours ago
unknown
unknown
22654 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. We use this to do the general case in #22656. --- I was uneasy about doing a special case first, but hopefully this short complex deserves to exist in its own right, since it's a more convenient expression for cores-coinf in the `S`-trivial case than a complex ending with `H₁(G ⧸ S, A_S)`... - [ ] depends on: #22651 - [ ] depends on: #22652 - [x] depends on: #21732 - [ ] depends on: #21733 - [ ] depends on: #21735 - [ ] depends on: #21736 - [ ] depends on: #21738 - [ ] depends on: #21740 - [ ] depends on: #21752 - [ ] depends on: #21754 - [ ] depends on: #21755 - [ ] depends on: #21757 - [ ] depends on: #21759 - [ ] depends on: #21763 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-algebra merge-conflict blocked-by-other-PR
label:t-algebra$
3384/965 Mathlib.lean,Mathlib/Algebra/BigOperators/Fin.lean,Mathlib/CategoryTheory/Action/Basic.lean,Mathlib/CategoryTheory/Action/Concrete.lean,Mathlib/CategoryTheory/Action/Monoidal.lean,Mathlib/CategoryTheory/Monoidal/Types/Basic.lean,Mathlib/Data/Finsupp/Basic.lean,Mathlib/GroupTheory/QuotientGroup/Defs.lean,Mathlib/LinearAlgebra/Finsupp/Defs.lean,Mathlib/RepresentationTheory/Basic.lean,Mathlib/RepresentationTheory/Coinvariants.lean,Mathlib/RepresentationTheory/GroupCohomology/Basic.lean,Mathlib/RepresentationTheory/GroupCohomology/Resolution.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/Basic.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/Functoriality.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/Hilbert90.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/LowDegree.lean,Mathlib/RepresentationTheory/Homological/GroupHomology/Basic.lean,Mathlib/RepresentationTheory/Homological/GroupHomology/Functoriality.lean,Mathlib/RepresentationTheory/Homological/GroupHomology/LowDegree.lean,Mathlib/RepresentationTheory/Homological/Resolution.lean,Mathlib/RepresentationTheory/Invariants.lean,Mathlib/RepresentationTheory/Rep.lean 23 n/a ['101damnations', 'acmepjz', 'github-actions', 'mathlib4-dependent-issues-bot'] nobody
0-41042
11 hours ago
unknown
unknown
21766 101damnations
author:101damnations
feat(RepresentationTheory/Homological/GroupHomology/LongExactSequence): specialise LES API to low degree group homology Given a commutative ring `k` and a group `G`, this file shows that a short exact sequence of `k`-linear `G`-representations `0 ⟶ X₁ ⟶ X₂ ⟶ X₃ ⟶ 0` induces a short exact sequence of complexes of inhomogeneous chains `0 ⟶ C(X₁) ⟶ C(X₂) ⟶ C(X₃) ⟶ 0`, where `Hₙ(C(Xᵢ))` is the `n`th group homology of `Xᵢ`. This allows us to specialize API about long exact sequences to group homology; in this PR we focus on degrees `n = 0, 1, 2`. --- - [x] depends on: #21652 - [x] depends on: #21732 - [ ] depends on: #21733 - [ ] depends on: #21735 - [ ] depends on: #21736 - [ ] depends on: #21738 - [ ] depends on: #21740 - [ ] depends on: #21752 - [ ] depends on: #21754 - [ ] depends on: #21755 - [ ] depends on: #21757 - [ ] depends on: #21759 - [ ] depends on: #21763 - [ ] depends on: #21764 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict blocked-by-other-PR
label:t-algebra$
3645/1178 Mathlib.lean,Mathlib/Algebra/BigOperators/Fin.lean,Mathlib/Algebra/Homology/ConcreteCategory.lean,Mathlib/Algebra/Homology/HomologySequence.lean,Mathlib/Algebra/Homology/ShortComplex/ModuleCat.lean,Mathlib/Algebra/Homology/ShortComplex/SnakeLemma.lean,Mathlib/CategoryTheory/Action/Basic.lean,Mathlib/CategoryTheory/Action/Concrete.lean,Mathlib/CategoryTheory/Action/Continuous.lean,Mathlib/CategoryTheory/Action/Limits.lean,Mathlib/CategoryTheory/Action/Monoidal.lean,Mathlib/CategoryTheory/Galois/Action.lean,Mathlib/CategoryTheory/Galois/EssSurj.lean,Mathlib/CategoryTheory/Galois/Examples.lean,Mathlib/CategoryTheory/Galois/Full.lean,Mathlib/CategoryTheory/Monoidal/Types/Basic.lean,Mathlib/Data/Fin/Tuple/Basic.lean,Mathlib/Data/Finsupp/Basic.lean,Mathlib/LinearAlgebra/Finsupp/Defs.lean,Mathlib/LinearAlgebra/Finsupp/Pi.lean,Mathlib/RepresentationTheory/Basic.lean,Mathlib/RepresentationTheory/Character.lean,Mathlib/RepresentationTheory/Coinvariants.lean,Mathlib/RepresentationTheory/FDRep.lean,Mathlib/RepresentationTheory/GroupCohomology/Basic.lean,Mathlib/RepresentationTheory/GroupCohomology/Resolution.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/Basic.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/Hilbert90.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/LowDegree.lean,Mathlib/RepresentationTheory/Homological/GroupHomology/Basic.lean,Mathlib/RepresentationTheory/Homological/GroupHomology/Functoriality.lean,Mathlib/RepresentationTheory/Homological/GroupHomology/LongExactSequence.lean,Mathlib/RepresentationTheory/Homological/GroupHomology/LowDegree.lean,Mathlib/RepresentationTheory/Homological/Resolution.lean,Mathlib/RepresentationTheory/Invariants.lean,Mathlib/RepresentationTheory/Rep.lean 36 n/a ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
0-41011
11 hours ago
unknown
unknown
21764 101damnations
author:101damnations
feat(RepresentationTheory/Homological/GroupHomology/LongExactSequence): specialise LES API to group homology Given a commutative ring `k` and a group `G`, this PR shows that a short exact sequence of `k`-linear `G`-representations `0 ⟶ X₁ ⟶ X₂ ⟶ X₃ ⟶ 0` induces a short exact sequence of complexes of inhomogeneous chains `0 ⟶ C(X₁) ⟶ C(X₂) ⟶ C(X₃) ⟶ 0`, where `Hₙ(C(Xᵢ))` is the `n`th group homology of `Xᵢ`. This allows us to specialize API about long exact sequences to group homology. --- - [x] depends on: #21652 - [x] depends on: #21732 - [ ] depends on: #21733 - [ ] depends on: #21735 - [ ] depends on: #21736 - [ ] depends on: #21738 - [ ] depends on: #21740 - [ ] depends on: #21752 - [ ] depends on: #21754 - [ ] depends on: #21755 - [ ] depends on: #21757 - [ ] depends on: #21759 - [ ] depends on: #21763 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict blocked-by-other-PR
label:t-algebra$
3449/1178 Mathlib.lean,Mathlib/Algebra/BigOperators/Fin.lean,Mathlib/Algebra/Homology/ConcreteCategory.lean,Mathlib/Algebra/Homology/HomologySequence.lean,Mathlib/Algebra/Homology/ShortComplex/ModuleCat.lean,Mathlib/Algebra/Homology/ShortComplex/SnakeLemma.lean,Mathlib/CategoryTheory/Action/Basic.lean,Mathlib/CategoryTheory/Action/Concrete.lean,Mathlib/CategoryTheory/Action/Continuous.lean,Mathlib/CategoryTheory/Action/Limits.lean,Mathlib/CategoryTheory/Action/Monoidal.lean,Mathlib/CategoryTheory/Galois/Action.lean,Mathlib/CategoryTheory/Galois/EssSurj.lean,Mathlib/CategoryTheory/Galois/Examples.lean,Mathlib/CategoryTheory/Galois/Full.lean,Mathlib/CategoryTheory/Monoidal/Types/Basic.lean,Mathlib/Data/Fin/Tuple/Basic.lean,Mathlib/Data/Finsupp/Basic.lean,Mathlib/LinearAlgebra/Finsupp/Defs.lean,Mathlib/LinearAlgebra/Finsupp/Pi.lean,Mathlib/RepresentationTheory/Basic.lean,Mathlib/RepresentationTheory/Character.lean,Mathlib/RepresentationTheory/Coinvariants.lean,Mathlib/RepresentationTheory/FDRep.lean,Mathlib/RepresentationTheory/GroupCohomology/Basic.lean,Mathlib/RepresentationTheory/GroupCohomology/Resolution.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/Basic.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/Hilbert90.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/LowDegree.lean,Mathlib/RepresentationTheory/Homological/GroupHomology/Basic.lean,Mathlib/RepresentationTheory/Homological/GroupHomology/Functoriality.lean,Mathlib/RepresentationTheory/Homological/GroupHomology/LongExactSequence.lean,Mathlib/RepresentationTheory/Homological/GroupHomology/LowDegree.lean,Mathlib/RepresentationTheory/Homological/Resolution.lean,Mathlib/RepresentationTheory/Invariants.lean,Mathlib/RepresentationTheory/Rep.lean 36 n/a ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
0-41010
11 hours ago
unknown
unknown
21763 101damnations
author:101damnations
feat(RepresentationTheory/Homological/GroupHomology/Functoriality): low degree functoriality maps Given a commutative ring `k`, a group homomorphism `f : G →* H`, a `k`-linear `G`-representation `A`, a `k`-linear `H`-representation `B`, and a representation morphism `A ⟶ Res(f)(B)`, we get a chain map `inhomogeneousChains A ⟶ inhomogeneousChains B` and hence maps on cohomology `Hₙ(G, A) ⟶ Hₙ(H, B)`. This PR provides specialised API for these maps in low degree. A future PR will add support for switching resolution. --- - [x] depends on: #21652 - [x] depends on: #21732 - [ ] depends on: #21733 - [ ] depends on: #21735 - [ ] depends on: #21736 - [ ] depends on: #21738 - [ ] depends on: #21740 - [ ] depends on: #21752 - [ ] depends on: #21754 - [ ] depends on: #21755 - [ ] depends on: #21757 - [ ] depends on: #21759 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict blocked-by-other-PR
label:t-algebra$
3215/1172 Mathlib.lean,Mathlib/Algebra/BigOperators/Fin.lean,Mathlib/CategoryTheory/Action/Basic.lean,Mathlib/CategoryTheory/Action/Concrete.lean,Mathlib/CategoryTheory/Action/Continuous.lean,Mathlib/CategoryTheory/Action/Limits.lean,Mathlib/CategoryTheory/Action/Monoidal.lean,Mathlib/CategoryTheory/Galois/Action.lean,Mathlib/CategoryTheory/Galois/EssSurj.lean,Mathlib/CategoryTheory/Galois/Examples.lean,Mathlib/CategoryTheory/Galois/Full.lean,Mathlib/CategoryTheory/Monoidal/Types/Basic.lean,Mathlib/Data/Fin/Tuple/Basic.lean,Mathlib/Data/Finsupp/Basic.lean,Mathlib/LinearAlgebra/Finsupp/Defs.lean,Mathlib/RepresentationTheory/Basic.lean,Mathlib/RepresentationTheory/Character.lean,Mathlib/RepresentationTheory/Coinvariants.lean,Mathlib/RepresentationTheory/FDRep.lean,Mathlib/RepresentationTheory/GroupCohomology/Basic.lean,Mathlib/RepresentationTheory/GroupCohomology/Resolution.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/Basic.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/Hilbert90.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/LowDegree.lean,Mathlib/RepresentationTheory/Homological/GroupHomology/Basic.lean,Mathlib/RepresentationTheory/Homological/GroupHomology/Functoriality.lean,Mathlib/RepresentationTheory/Homological/GroupHomology/LowDegree.lean,Mathlib/RepresentationTheory/Homological/Resolution.lean,Mathlib/RepresentationTheory/Invariants.lean,Mathlib/RepresentationTheory/Rep.lean 30 n/a ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
0-41009
11 hours ago
unknown
unknown
21762 101damnations
author:101damnations
feat(RepresentationTheory/Homological/GroupHomology/LowDegree): `H₁(G, A) ≃+ Gᵃᵇ ⊗[ℤ] A` when `A` is trivial This PR defines an isomorphism `H₁(G, A) ≃+ Gᵃᵇ ⊗[ℤ] A` when the `G`-representation on `A` is trivial. --- - [x] depends on: #21652 - [x] depends on: #21732 - [x] depends on: #21733 - [ ] depends on: #21735 - [ ] depends on: #21736 - [ ] depends on: #21738 - [ ] depends on: #21740 - [ ] depends on: #21752 - [ ] depends on: #21755 - [ ] depends on: #21757 - [ ] depends on: #21759 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict blocked-by-other-PR
label:t-algebra$
2793/1172 Mathlib.lean,Mathlib/Algebra/BigOperators/Fin.lean,Mathlib/CategoryTheory/Action/Basic.lean,Mathlib/CategoryTheory/Action/Concrete.lean,Mathlib/CategoryTheory/Action/Continuous.lean,Mathlib/CategoryTheory/Action/Limits.lean,Mathlib/CategoryTheory/Action/Monoidal.lean,Mathlib/CategoryTheory/Galois/Action.lean,Mathlib/CategoryTheory/Galois/EssSurj.lean,Mathlib/CategoryTheory/Galois/Examples.lean,Mathlib/CategoryTheory/Galois/Full.lean,Mathlib/CategoryTheory/Monoidal/Types/Basic.lean,Mathlib/LinearAlgebra/Finsupp/Defs.lean,Mathlib/RepresentationTheory/Basic.lean,Mathlib/RepresentationTheory/Character.lean,Mathlib/RepresentationTheory/Coinvariants.lean,Mathlib/RepresentationTheory/FDRep.lean,Mathlib/RepresentationTheory/GroupCohomology/Basic.lean,Mathlib/RepresentationTheory/GroupCohomology/Resolution.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/Basic.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/Hilbert90.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/LowDegree.lean,Mathlib/RepresentationTheory/Homological/GroupHomology/Basic.lean,Mathlib/RepresentationTheory/Homological/GroupHomology/LowDegree.lean,Mathlib/RepresentationTheory/Homological/Resolution.lean,Mathlib/RepresentationTheory/Invariants.lean,Mathlib/RepresentationTheory/Rep.lean 27 n/a ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
0-41008
11 hours ago
unknown
unknown
21759 101damnations
author:101damnations
feat(RepresentationTheory/Homological/GroupHomology/LowDegree): Identify `groupHomology A n` with `Hn A` for `n = 0, 1, 2` This PR gives isomorphisms between `groupHomology A n` (defined as the `n`th homology of the complex of inhomogeneous chains of `A`, whose `n`th object is `Gⁿ →₀ A`, and `Hn A` (defined more minimally and explicitly) for `n = 0, 1, 2`. We do the same for cycles. --- - [x] depends on: #21652 - [x] depends on: #21732 - [ ] depends on: #21733 - [ ] depends on: #21735 - [ ] depends on: #21736 - [ ] depends on: #21738 - [ ] depends on: #21740 - [ ] depends on: #21752 - [ ] depends on: #21755 - [ ] depends on: #21757 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict blocked-by-other-PR
label:t-algebra$
2719/1172 Mathlib.lean,Mathlib/Algebra/BigOperators/Fin.lean,Mathlib/CategoryTheory/Action/Basic.lean,Mathlib/CategoryTheory/Action/Concrete.lean,Mathlib/CategoryTheory/Action/Continuous.lean,Mathlib/CategoryTheory/Action/Limits.lean,Mathlib/CategoryTheory/Action/Monoidal.lean,Mathlib/CategoryTheory/Galois/Action.lean,Mathlib/CategoryTheory/Galois/EssSurj.lean,Mathlib/CategoryTheory/Galois/Examples.lean,Mathlib/CategoryTheory/Galois/Full.lean,Mathlib/CategoryTheory/Monoidal/Types/Basic.lean,Mathlib/LinearAlgebra/Finsupp/Defs.lean,Mathlib/RepresentationTheory/Basic.lean,Mathlib/RepresentationTheory/Character.lean,Mathlib/RepresentationTheory/Coinvariants.lean,Mathlib/RepresentationTheory/FDRep.lean,Mathlib/RepresentationTheory/GroupCohomology/Basic.lean,Mathlib/RepresentationTheory/GroupCohomology/Resolution.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/Basic.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/Hilbert90.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/LowDegree.lean,Mathlib/RepresentationTheory/Homological/GroupHomology/Basic.lean,Mathlib/RepresentationTheory/Homological/GroupHomology/LowDegree.lean,Mathlib/RepresentationTheory/Homological/Resolution.lean,Mathlib/RepresentationTheory/Invariants.lean,Mathlib/RepresentationTheory/Rep.lean 27 n/a ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
0-41007
11 hours ago
unknown
unknown
21757 101damnations
author:101damnations
feat(RepresentationTheory/Homological/GroupHomology/LowDegree): add `IsOneCycle` predicate and friends Given an additive abelian group `A` with an appropriate scalar action of `G`, we provide support for turning a finsupp `f : G →₀ A` satisfying the 1-cycle identity into an element of the `oneCycles` of the representation on `A` corresponding to the scalar action. We also do this for 0-boundaries, 1-boundaries, 2-cycles and 2-boundaries. We follow the structure of `RepresentationTheory.Homological.GroupCohomology.LowDegree`. --- - [x] depends on: #21652 - [x] depends on: #21732 - [ ] depends on: #21733 - [ ] depends on: #21735 - [ ] depends on: #21736 - [ ] depends on: #21738 - [ ] depends on: #21740 - [ ] depends on: #21752 - [ ] depends on: #21755 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict blocked-by-other-PR
label:t-algebra$
2442/1172 Mathlib.lean,Mathlib/Algebra/BigOperators/Fin.lean,Mathlib/CategoryTheory/Action/Basic.lean,Mathlib/CategoryTheory/Action/Concrete.lean,Mathlib/CategoryTheory/Action/Continuous.lean,Mathlib/CategoryTheory/Action/Limits.lean,Mathlib/CategoryTheory/Action/Monoidal.lean,Mathlib/CategoryTheory/Galois/Action.lean,Mathlib/CategoryTheory/Galois/EssSurj.lean,Mathlib/CategoryTheory/Galois/Examples.lean,Mathlib/CategoryTheory/Galois/Full.lean,Mathlib/CategoryTheory/Monoidal/Types/Basic.lean,Mathlib/LinearAlgebra/Finsupp/Defs.lean,Mathlib/RepresentationTheory/Basic.lean,Mathlib/RepresentationTheory/Character.lean,Mathlib/RepresentationTheory/Coinvariants.lean,Mathlib/RepresentationTheory/FDRep.lean,Mathlib/RepresentationTheory/GroupCohomology/Basic.lean,Mathlib/RepresentationTheory/GroupCohomology/Resolution.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/Basic.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/Hilbert90.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/LowDegree.lean,Mathlib/RepresentationTheory/Homological/GroupHomology/Basic.lean,Mathlib/RepresentationTheory/Homological/GroupHomology/LowDegree.lean,Mathlib/RepresentationTheory/Homological/Resolution.lean,Mathlib/RepresentationTheory/Invariants.lean,Mathlib/RepresentationTheory/Rep.lean 27 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
0-41007
11 hours ago
52-84569
1 month ago
0-422
7 minutes
21755 101damnations
author:101damnations
feat(RepresentationTheory/Homological/GroupHomology/LowDegree): API for(one/two)(Cycles/Boundaries) This PR is more API for low degree group homology, adding (one/two)(Cycles/Boundaries), following the structure of `RepresentationTheory.Homological.GroupCohomology.LowDegree`. --- - [x] depends on: #21652 - [x] depends on: #21732 - [ ] depends on: #21733 - [ ] depends on: #21735 - [ ] depends on: #21736 - [ ] depends on: #21738 - [ ] depends on: #21740 - [ ] depends on: #21752 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict blocked-by-other-PR
label:t-algebra$
2247/1172 Mathlib.lean,Mathlib/Algebra/BigOperators/Fin.lean,Mathlib/CategoryTheory/Action/Basic.lean,Mathlib/CategoryTheory/Action/Concrete.lean,Mathlib/CategoryTheory/Action/Continuous.lean,Mathlib/CategoryTheory/Action/Limits.lean,Mathlib/CategoryTheory/Action/Monoidal.lean,Mathlib/CategoryTheory/Galois/Action.lean,Mathlib/CategoryTheory/Galois/EssSurj.lean,Mathlib/CategoryTheory/Galois/Examples.lean,Mathlib/CategoryTheory/Galois/Full.lean,Mathlib/CategoryTheory/Monoidal/Types/Basic.lean,Mathlib/LinearAlgebra/Finsupp/Defs.lean,Mathlib/RepresentationTheory/Basic.lean,Mathlib/RepresentationTheory/Character.lean,Mathlib/RepresentationTheory/Coinvariants.lean,Mathlib/RepresentationTheory/FDRep.lean,Mathlib/RepresentationTheory/GroupCohomology/Basic.lean,Mathlib/RepresentationTheory/GroupCohomology/Resolution.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/Basic.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/Hilbert90.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/LowDegree.lean,Mathlib/RepresentationTheory/Homological/GroupHomology/Basic.lean,Mathlib/RepresentationTheory/Homological/GroupHomology/LowDegree.lean,Mathlib/RepresentationTheory/Homological/Resolution.lean,Mathlib/RepresentationTheory/Invariants.lean,Mathlib/RepresentationTheory/Rep.lean 27 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
0-41006
11 hours ago
52-84562
1 month ago
0-201
3 minutes
21754 101damnations
author:101damnations
feat(RepresentationTheory/Homological/GroupHomology/Functoriality): add functoriality Given a commutative ring `k`, a group homomorphism `f : G →* H`, a `k`-linear `G`-representation `A`, a `k`-linear `H`-representation `B`, and a representation morphism `A ⟶ Res(f)(B)`, we get a chain map `inhomogeneousChains A ⟶ inhomogeneousChains B` and hence maps on group homology `Hₙ(G, A) ⟶ Hₙ(H, B)`. A subsequent PR will add specialised API for low degree, and a future PR will add support for switching resolution. --- - [x] depends on: #21652 - [x] depends on: #21732 - [ ] depends on: #21733 - [ ] depends on: #21735 - [ ] depends on: #21736 - [ ] depends on: #21738 - [ ] depends on: #21740 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict blocked-by-other-PR
label:t-algebra$
1989/1172 Mathlib.lean,Mathlib/Algebra/BigOperators/Fin.lean,Mathlib/CategoryTheory/Action/Basic.lean,Mathlib/CategoryTheory/Action/Concrete.lean,Mathlib/CategoryTheory/Action/Continuous.lean,Mathlib/CategoryTheory/Action/Limits.lean,Mathlib/CategoryTheory/Action/Monoidal.lean,Mathlib/CategoryTheory/Galois/Action.lean,Mathlib/CategoryTheory/Galois/EssSurj.lean,Mathlib/CategoryTheory/Galois/Examples.lean,Mathlib/CategoryTheory/Galois/Full.lean,Mathlib/CategoryTheory/Monoidal/Types/Basic.lean,Mathlib/Data/Fin/Tuple/Basic.lean,Mathlib/Data/Finsupp/Basic.lean,Mathlib/LinearAlgebra/Finsupp/Defs.lean,Mathlib/RepresentationTheory/Basic.lean,Mathlib/RepresentationTheory/Character.lean,Mathlib/RepresentationTheory/Coinvariants.lean,Mathlib/RepresentationTheory/FDRep.lean,Mathlib/RepresentationTheory/GroupCohomology/Basic.lean,Mathlib/RepresentationTheory/GroupCohomology/Resolution.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/Basic.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/Hilbert90.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/LowDegree.lean,Mathlib/RepresentationTheory/Homological/GroupHomology/Basic.lean,Mathlib/RepresentationTheory/Homological/GroupHomology/Functoriality.lean,Mathlib/RepresentationTheory/Homological/Resolution.lean,Mathlib/RepresentationTheory/Invariants.lean,Mathlib/RepresentationTheory/Rep.lean 29 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
0-41005
11 hours ago
52-84554
1 month ago
0-219
3 minutes
21752 101damnations
author:101damnations
feat(RepresentationTheory/Homological/GroupHomology/LowDegree): simpler expressions for differentials The first part of a file giving simpler expressions for group homology in low degree, following the structure of `RepresentationTheory.Homological.GroupCohomology.LowDegree`. --- - [x] depends on: #21652 - [x] depends on: #21732 - [ ] depends on: #21733 - [ ] depends on: #21735 - [ ] depends on: #21736 - [ ] depends on: #21738 - [ ] depends on: #21740 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) file-removed large-import t-algebra merge-conflict blocked-by-other-PR
label:t-algebra$
1991/961 Mathlib.lean,Mathlib/Algebra/BigOperators/Fin.lean,Mathlib/CategoryTheory/Action/Basic.lean,Mathlib/CategoryTheory/Action/Concrete.lean,Mathlib/CategoryTheory/Action/Monoidal.lean,Mathlib/CategoryTheory/Monoidal/Types/Basic.lean,Mathlib/RepresentationTheory/Basic.lean,Mathlib/RepresentationTheory/Coinvariants.lean,Mathlib/RepresentationTheory/GroupCohomology/Basic.lean,Mathlib/RepresentationTheory/GroupCohomology/Resolution.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/Basic.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/Functoriality.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/Hilbert90.lean,Mathlib/RepresentationTheory/Homological/GroupCohomology/LowDegree.lean,Mathlib/RepresentationTheory/Homological/GroupHomology/Basic.lean,Mathlib/RepresentationTheory/Homological/GroupHomology/LowDegree.lean,Mathlib/RepresentationTheory/Homological/Resolution.lean,Mathlib/RepresentationTheory/Invariants.lean,Mathlib/RepresentationTheory/Rep.lean 19 n/a ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
0-41004
11 hours ago
unknown
unknown
25311 101damnations
author:101damnations
feat(RepresentationTheory/GroupCohomology): long exact sequences (again) --- - [ ] depends on: #25310 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict blocked-by-other-PR WIP
label:t-algebra$
706/542 Mathlib.lean,Mathlib/Algebra/Homology/ConcreteCategory.lean,Mathlib/Algebra/Homology/HomologySequence.lean,Mathlib/Algebra/Homology/ShortComplex/SnakeLemma.lean,Mathlib/LinearAlgebra/Pi.lean,Mathlib/RepresentationTheory/GroupCohomology/Basic.lean,Mathlib/RepresentationTheory/GroupCohomology/Functoriality.lean,Mathlib/RepresentationTheory/GroupCohomology/Hilbert90.lean,Mathlib/RepresentationTheory/GroupCohomology/LongExactSequence.lean,Mathlib/RepresentationTheory/GroupCohomology/LowDegree.lean 10 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
0-35790
9 hours ago
0-35791
9 hours ago
0-10
10 seconds
24822 CBirkbeck
author:CBirkbeck
feat: define the Eisenstein Series E2 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-number-theory merge-conflict 159/0 Mathlib/NumberTheory/ModularForms/EisensteinSeries/E2.lean,Mathlib/NumberTheory/ModularForms/EisensteinSeries/UniformConvergence.lean 2 2 ['github-actions', 'leanprover-community-bot-assistant'] nobody
0-22053
6 hours ago
0-22055
6 hours ago
0-0
0 seconds
24962 loefflerd
author:loefflerd
WIP towards Hecke bound for q-expansions The aim of this PR is to prove various statements about boundedness properties of modular forms. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-number-theory merge-conflict WIP 793/139 Mathlib.lean,Mathlib/NumberTheory/ModularForms/Bounds.lean,Mathlib/NumberTheory/ModularForms/CongruenceSubgroups.lean,Mathlib/NumberTheory/ModularForms/EisensteinSeries/IsBoundedAtImInfty.lean,Mathlib/NumberTheory/ModularForms/Identities.lean,Mathlib/NumberTheory/ModularForms/LevelOne.lean,Mathlib/NumberTheory/ModularForms/Petersson.lean,Mathlib/NumberTheory/ModularForms/QExpansion.lean 8 3 ['github-actions', 'leanprover-community-bot-assistant'] nobody
0-21930
6 hours ago
0-21932
6 hours ago
0-1
1 second
25393 CBirkbeck
author:CBirkbeck
feat: Add more Summability results needed for Eisenstein series. We add results about the summability of the term (c z + d)^-k that are needed for Eisenstein series (such as E2). --- - [ ] depends on: #25443 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-number-theory merge-conflict WIP 248/134 Mathlib.lean,Mathlib/Analysis/Asymptotics/Defs.lean,Mathlib/Analysis/Complex/Asymptotics.lean,Mathlib/Analysis/Normed/Group/Bounded.lean,Mathlib/NumberTheory/ModularForms/EisensteinSeries/IsBoundedAtImInfty.lean,Mathlib/NumberTheory/ModularForms/EisensteinSeries/Summable.lean,Mathlib/NumberTheory/ModularForms/EisensteinSeries/UniformConvergence.lean 7 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
0-21536
5 hours ago
0-21538
5 hours ago
1-10522
1 day
25448 CBirkbeck
author:CBirkbeck
Add the Mittag-Leffler expansion for cotangent We prove the Mittag-Leffler series expansion for `cot(pi z)`, which says ``` theorem cot_series_rep {z : ℂ} (hz : z ∈ ℂ_ℤ) : π * Complex.cot (π * z) = 1 / z + ∑' n : ℕ+, (1 / ((z : ℂ) - n) + 1 / (z + n)) ``` --- - [x] depends on: #25446 - [ ] depends on: #25393 - [ ] depends on: #25443 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import merge-conflict blocked-by-other-PR WIP 430/137 Mathlib.lean,Mathlib/Analysis/Asymptotics/Defs.lean,Mathlib/Analysis/Complex/Asymptotics.lean,Mathlib/Analysis/Complex/IntegerCompl.lean,Mathlib/Analysis/Complex/LocallyUniformLimit.lean,Mathlib/Analysis/Normed/Group/Bounded.lean,Mathlib/Analysis/SpecialFunctions/Log/Summable.lean,Mathlib/Analysis/SpecialFunctions/Trigonometric/Cotangent.lean,Mathlib/NumberTheory/ModularForms/EisensteinSeries/IsBoundedAtImInfty.lean,Mathlib/NumberTheory/ModularForms/EisensteinSeries/Summable.lean,Mathlib/NumberTheory/ModularForms/EisensteinSeries/UniformConvergence.lean 11 4 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
0-21535
5 hours ago
0-21537
5 hours ago
0-1521
25 minutes
25219 Multramate
author:Multramate
feat(AlgebraicGeometry/EllipticCurve): generalise nonsingular condition --- - [ ] depends on: #24593 - [ ] depends on: #25323 - [x] depends on: #25378 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra t-algebraic-geometry awaiting-CI merge-conflict blocked-by-other-PR WIP
label:t-algebra$
1527/1274 Mathlib/Algebra/Module/PID.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Affine/Basic.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Affine/Formula.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Affine/Point.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Jacobian/Basic.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Jacobian/Formula.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Jacobian/Point.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Projective/Basic.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Projective/Formula.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Projective/Point.lean,Mathlib/RingTheory/DedekindDomain/AdicValuation.lean,Mathlib/RingTheory/Ideal/Maps.lean,Mathlib/RingTheory/Ideal/Span.lean 13 5 ['github-actions', 'kckennylau', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
0-7337
2 hours ago
2-57062
2 days ago
0-1
1 second
24789 Ruben-VandeVelde
author:Ruben-VandeVelde
chore: move Algebra.Group.Hom.End to Algebra.Ring --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import t-algebra merge-conflict awaiting-author
label:t-algebra$
55/50 Mathlib.lean,Mathlib/Algebra/Group/Hom/End.lean,Mathlib/Algebra/Group/Hom/Instances.lean,Mathlib/Algebra/Module/End.lean,Mathlib/Algebra/Ring/Hom/End.lean 5 6 ['Ruben-VandeVelde', 'YaelDillies', 'eric-wieser', 'github-actions', 'leanprover-community-bot-assistant'] nobody
0-5911
1 hour ago
0-5913
1 hour ago
0-1530
25 minutes
25264 linesthatinterlace
author:linesthatinterlace
feat: add elementary lifts for `OneHom`, `MulHom`, `MonoidHom` and `RingHom`. Adds `liftRight` and `liftLeft` constructions for `OneHom`, `MulHom` and `MonoidHom`. --- The plan is to implement `Units.liftRight` and possibly other "lift"-style monoid constructions (e.g. `liftOfRightInverse`) using these. This should probably be in a future PR but I could consider adding it to this one once the initial changes are stable. Note that these constructions are added relatively deep as they do not need much in the way of pre-requisites. [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict
label:t-algebra$
412/11 Mathlib/Algebra/Group/Hom/Basic.lean,Mathlib/Algebra/Group/Hom/Defs.lean,Mathlib/Algebra/Ring/Hom/Basic.lean,Mathlib/Algebra/Ring/Hom/Defs.lean 4 7 ['eric-wieser', 'github-actions', 'leanprover-community-bot-assistant', 'linesthatinterlace'] nobody
0-5787
1 hour ago
0-5789
1 hour ago
12-4669
12 days
25296 linesthatinterlace
author:linesthatinterlace
feat: Add high-level generalizations from `MonoidHom` lifts Replaces high-level definitions of `liftOfRightInverse` etc. with low-level equivalents. --- - [ ] depends on: #25290 - [ ] depends on: #25264 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra merge-conflict blocked-by-other-PR
label:t-algebra$
1256/168 Mathlib/Algebra/Category/Ring/FinitePresentation.lean,Mathlib/Algebra/Group/Equiv/Basic.lean,Mathlib/Algebra/Group/Hom/Basic.lean,Mathlib/Algebra/Group/Hom/Defs.lean,Mathlib/Algebra/Group/Subgroup/Basic.lean,Mathlib/Algebra/Polynomial/Div.lean,Mathlib/Algebra/Polynomial/Roots.lean,Mathlib/Algebra/Ring/Equiv.lean,Mathlib/Algebra/Ring/Hom/Basic.lean,Mathlib/Algebra/Ring/Hom/Defs.lean,Mathlib/Data/Int/Cast/Lemmas.lean,Mathlib/Data/ZMod/Basic.lean,Mathlib/NumberTheory/ClassNumber/Finite.lean,Mathlib/NumberTheory/DirichletCharacter/Basic.lean,Mathlib/RingTheory/Ideal/Maps.lean,Mathlib/RingTheory/Polynomial/Content.lean,Mathlib/RingTheory/RootsOfUnity/Minpoly.lean 17 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
0-5663
1 hour ago
0-5665
1 hour ago
0-688
11 minutes

Other lists of PRs

Some other lists of PRs which could be useful:

PRs with non-conforming titles

Number Author Title Description Labels +/- Modified files (first 100) 📝 💬 All users who commented or reviewed Assignee(s) Updated Last status change total time in review
25173 Timeroot
author:Timeroot
"Junk value" test file Add to MathlibTest a file that documents junk values of many functions, and explains some of their motivations and gotchas. --- Based on the conversation [on Zulip](https://leanprover.zulipchat.com/#narrow/channel/113488-general/topic/Documenting.20lean.20pitfalls.3A.20feedback.20requested/near/520155520). [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 362/2 Mathlib/Data/Nat/Find.lean,MathlibTest/Junk.lean 2 15 ['Timeroot', 'github-actions', 'plp127'] nobody
11-84537
11 days ago
15-59398
15 days ago
15-59382
15 days
25474 adomani
author:adomani
test for .lean/.md check A test PR for #25473. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) file-removed 10/1 .github/workflows/lint_and_suggest_pr.yml,Mathlib.lean,Mathlib/NumberTheory/NumberField/CMField.Lean 3 1 ['github-actions'] nobody
4-36516
4 days ago
4-37849
4 days ago
4-37907
4 days
25459 emilyriehl
author:emilyriehl
Feat(CategoryTheory): terminal categories with an application to hoFunctor Some preliminary API around terminal categories is developed with an application for the infinity-cosmos project: proving that the homotopy category functor preserves terminal objects. We also include proofs that `[0]` is terminal in the simplex category and `Δ[0]` is the terminal simplicial set. Co-authored by [Robin Carlier](robin.carlier@ens-lyon.fr), [Adam Topaz](topaz@ualberta.ca), and [Zeyi Zhao](zzhao95@jh.edu). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) infinity-cosmos large-import t-category-theory 178/3 Mathlib.lean,Mathlib/AlgebraicTopology/SimplexCategory/Basic.lean,Mathlib/AlgebraicTopology/SimplicialSet/HomotopyCat.lean,Mathlib/AlgebraicTopology/SimplicialSet/Monoidal.lean,Mathlib/CategoryTheory/Category/Cat/Terminal.lean,Mathlib/CategoryTheory/Category/ReflQuiv.lean,Mathlib/CategoryTheory/Quotient.lean 7 3 ['emilyriehl', 'github-actions', 'jcommelin'] nobody
2-47711
2 days ago
4-23991
4 days ago
4-81274
4 days
25608 TOMILO87
author:TOMILO87
Add Beta distribution feat(Probability/Distributions): add Beta distribution Add the Beta distribution to the probability distributions in mathlib4. This implementation includes: - Definition of the Beta function over the reals - The probability density function (PDF) of the Beta distribution - Proof that the PDF integrates to 1 - Various lemmas about measurability and positivity properties The Beta distribution is a family of continuous probability distributions defined on the interval [0, 1] parametrized by two positive shape parameters, α and β, that control the shape of the distribution. The implementation follows a similar structure to other distributions in mathlib4, particularly the Gamma distribution, adapting the approach to the specific properties of the Beta distribution. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor t-measure-probability 257/0 Mathlib.lean,Mathlib/Probability/Distributions/Beta.lean 2 1 ['github-actions'] nobody
0-76007
21 hours ago
0-76019
21 hours ago
0-76075
21 hours
25470 mans0954
author:mans0954
Low order roots of unity Compute some low order roots of unity. [Zulip discussion](https://leanprover.zulipchat.com/#narrow/channel/116395-maths/topic/roots.20of.20unity.20-.20computing.20low.20degree/with/520523576) Cubic case contributed by @MichaelStollBayreuth See also: #25215, #24828 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) t-algebra
label:t-algebra$
182/0 Mathlib/Algebra/CharP/Invertible.lean,Mathlib/RingTheory/RootsOfUnity/Complex.lean 2 1 ['github-actions'] nobody
0-46136
12 hours ago
0-46136
12 hours ago
2-75320
2 days
23644 JovanGerb
author:JovanGerb
Lean pr testing 7804 Testing an optimization in `simp` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict 4/4 lake-manifest.json,lakefile.lean,lean-toolchain 3 3 ['github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot'] nobody
4-29888
4 days ago
66-75572
2 months ago
0-2933
48 minutes
24808 JovanGerb
author:JovanGerb
lean pr testing 8294 Testing a cache optimization in `isDefEq`, to avoid exponential blowup during unification. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict 243/98 Mathlib.lean,Mathlib/Algebra/BigOperators/Group/Finset/Basic.lean,Mathlib/Algebra/BigOperators/Group/Finset/Preimage.lean,Mathlib/Algebra/BigOperators/Intervals.lean,Mathlib/Algebra/Group/Submonoid/Basic.lean,Mathlib/Algebra/GroupWithZero/Basic.lean,Mathlib/Algebra/GroupWithZero/Defs.lean,Mathlib/Algebra/GroupWithZero/NeZero.lean,Mathlib/Algebra/Homology/DifferentialObject.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Affine/Formula.lean,Mathlib/AlgebraicGeometry/EllipticCurve/Affine/Point.lean,Mathlib/Analysis/Complex/ValueDistribution/CharacteristicFunction.lean,Mathlib/Analysis/InnerProductSpace/Spectrum.lean,Mathlib/Analysis/LConvolution.lean,Mathlib/Analysis/NormedSpace/Alternating/Curry.lean,Mathlib/CategoryTheory/Limits/VanKampen.lean,Mathlib/Data/Finset/Fold.lean,Mathlib/Data/Finset/Image.lean,Mathlib/Data/Int/Init.lean,Mathlib/Data/Matrix/Mul.lean,Mathlib/Data/Nat/Factorization/Basic.lean,Mathlib/Data/Set/Function.lean,Mathlib/Data/Set/Image.lean,Mathlib/Data/Vector/MapLemmas.lean,Mathlib/Data/ZMod/Basic.lean,Mathlib/MeasureTheory/Group/Convolution.lean,Mathlib/MeasureTheory/Group/IntegralConvolution.lean,Mathlib/NumberTheory/ArithmeticFunction.lean,Mathlib/NumberTheory/Divisors.lean,Mathlib/Probability/Distributions/Gaussian/Real.lean,Mathlib/Topology/Algebra/InfiniteSum/NatInt.lean,Shake/Main.lean,lake-manifest.json,lakefile.lean,lean-toolchain 35 21 ['JovanGerb', 'adomani', 'github-actions', 'leanprover-bot', 'leanprover-community-mathlib4-bot'] nobody
2-686
2 days ago
2-686
2 days ago
0-11360
3 hours

PRs without an area label

Number Author Title Description Labels +/- Modified files (first 100) 📝 💬 All users who commented or reviewed Assignee(s) Updated Last status change total time in review
25238 Hagb
author:Hagb
feat(Tactic/ComputeDegree): add support for scalar multiplication with different types It would be able to deal with `a • (X : R[X])` where `a : S` is in a different type `S` with `[SMulZeroClass S R]`. --- - [x] depends on: #25237 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor 17/5 Mathlib/Tactic/ComputeDegree.lean,MathlibTest/ComputeDegree.lean 2 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
12-56734
12 days ago
12-81177
12 days ago
12-83080
12 days
25253 Ruben-VandeVelde
author:Ruben-VandeVelde
feat: add AlgHom.natCard_of_splits --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 21/7 Mathlib/FieldTheory/PrimitiveElement.lean,Mathlib/FieldTheory/Separable.lean,Mathlib/SetTheory/Cardinal/Finite.lean 3 1 ['github-actions'] nobody
12-43025
12 days ago
12-43107
12 days ago
12-43091
12 days
25327 YaelDillies
author:YaelDillies
feat: `F.obj M` is a commutative monoid object if `M` is From Toric --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) toric 11/3 Mathlib/CategoryTheory/Monoidal/CommMon_.lean,Mathlib/CategoryTheory/Monoidal/Mon_.lean 2 1 ['github-actions'] nobody
7-35334
7 days ago
9-34472
9 days ago
9-34465
9 days
25407 adomani
author:adomani
feat: check that the mathlib options exist This PR adds a simple check that all the options mentioned in `mathlibStandardSet` exist (at least, the ones that do exist!). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) maintainer-merge 18/0 Mathlib/Init.lean 1 5 ['adomani', 'github-actions', 'grunweg'] nobody
4-85198
4 days ago
4-85198
4 days ago
5-82859
5 days
25484 VTrelat
author:VTrelat
feat(SetTheory/ZFC/Booleans): define Boolean algebra in ZFC Extend the model of ZFC with Boolean algebra: - define a set 𝔹 of booleans - define a proper type `ZFBool` representing booleans - add theorems on usual algebraic properties of booleans - provide usual boolean notations like `⊤`, `⊥`, `∧`, `∨`, etc. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) - [ ] depends on: #25483 new-contributor blocked-by-other-PR 619/0 Mathlib/Data/Set/Prod.lean,Mathlib/SetTheory/ZFC/Basic.lean,Mathlib/SetTheory/ZFC/Booleans.lean 3 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
4-24128
4 days ago
4-24130
4 days ago
0-1523
25 minutes
25485 VTrelat
author:VTrelat
feat(SetTheory/ZFC/Naturals): define natural numbers in ZFC Extend the model of ZFC with naturals: - define a set `Nat` of naturals following the usual construction (∅, {∅}, {∅, {∅}}, ...) - define a proper type `ZFNat` representing naturals - add theorems on usual algebraic properties of naturals - provide a recursor and induction schemes to define/prove by induction --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) - [ ] depend on: #25483 new-contributor 2095/0 Mathlib/Data/Set/Prod.lean,Mathlib/SetTheory/ZFC/Basic.lean,Mathlib/SetTheory/ZFC/Booleans.lean,Mathlib/SetTheory/ZFC/Naturals.lean 4 1 ['github-actions'] nobody
4-22216
4 days ago
4-22281
4 days ago
4-22277
4 days
25488 VTrelat
author:VTrelat
feat(SetTheory/ZFC/Rationals): define rationals in ZFC Extend the model of ZFC with rationals: we define a proper type `ZFRat` representing integers based on pairs of `ZFInt` (enforcing the res to be nonzero) and following the usual construction of rationals. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) - [ ] depends on: #25483 - [ ] depends on: #25485 - [ ] depends on: #25486 new-contributor blocked-by-other-PR 2070/0 Mathlib/Data/Set/Prod.lean,Mathlib/SetTheory/ZFC/Basic.lean,Mathlib/SetTheory/ZFC/Booleans.lean,Mathlib/SetTheory/ZFC/Integers.lean,Mathlib/SetTheory/ZFC/Rationals.lean 5 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
4-19805
4 days ago
4-19807
4 days ago
0-1808
30 minutes
25486 VTrelat
author:VTrelat
feat(SetTheory/ZFC/Integers): define integers in ZFC Extend the model of ZFC with integers following the converse direction as for naturals. We first define a type and then build a set. We finally show that both representations have coercions in both direction: - define a proper type `ZFInt` representing integers based on `ZFNat × ZFNat` and following the usual construction of integers - add theorems on usual algebraic properties of integers - define a set `Int` and show that it matches-i.e. that it is isomorphic to-the type `ZFInt` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) - [ ] depends on: #25483 - [ ] depends on: #25485 new-contributor blocked-by-other-PR 2003/0 Mathlib/Data/Set/Prod.lean,Mathlib/SetTheory/ZFC/Basic.lean,Mathlib/SetTheory/ZFC/Booleans.lean,Mathlib/SetTheory/ZFC/Integers.lean 4 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
4-19803
4 days ago
4-19805
4 days ago
0-2067
34 minutes
25537 literandltx
author:literandltx
feat(number_theory/legendre_symbol): Add sqrt‐of‐residue theorems for p=4k+3 and p=8k+5 Add a new file `QuadraticResidueRoots.lean` under `Mathlib/NumberTheory/LegendreSymbol/` that proves two explicit “square-root of quadratic residue” theorems for primes of the specific form. - **`exists_sqrt_of_residue_mod4_eq3`** for primes `p = 4*k + 3` - **`exists_sqrt_of_residue_mod8_eq5`** for primes `p = 8*k + 5` It also introduces the helper lemmas `euler_criterion_traditional` and `legendreSym.at_two_mod8_eq_5`. Import lines in `Mathlib.lean` and `Mathlib/NumberTheory/LegendreSymbol/Basic.lean` have been updated accordingly. new-contributor 217/0 Mathlib.lean,Mathlib/NumberTheory/LegendreSymbol/Basic.lean,Mathlib/NumberTheory/LegendreSymbol/QuadraticReciprocity.lean,Mathlib/NumberTheory/LegendreSymbol/QuadraticResidueRoots.lean 4 0 [] nobody
3-19735
3 days ago
3-19735
3 days ago
0-0
0 seconds
25604 sgouezel
author:sgouezel
feat: make sure that the simp normal form of equiv-like classes pushes `symm` and `trans` to the right This follows the usual convention for coercions. See discussion at [#mathlib4 > simp normal form for symm and coercions @ 💬](https://leanprover.zulipchat.com/#narrow/channel/287929-mathlib4/topic/simp.20normal.20form.20for.20symm.20and.20coercions/near/522879475) For each equiv class, after the PR we should have lemmas like ```lean @[simp] lemma coe_toEquiv (e : G ≃+c[a, b] H) : ⇑e.toEquiv = e := rfl @[simp] lemma coe_symm_toEquiv (e : G ≃+c[a, b] H) : ⇑e.toEquiv.symm = e.symm := rfl @[simp] lemma toEquiv_symm (e : G ≃+c[a, b] H) : e.symm.toEquiv = e.toEquiv.symm := rfl @[simp] lemma toEquiv_trans (e₁ : G ≃+c[a, b] H) (e₂ : H ≃+c[b, c] K) : (e₁.trans e₂).toEquiv = e₁.toEquiv.trans e₂.toEquiv := rfl ``` The PR does not complete this task, because it would require killing the coercion from EquivLike classes to Equivs (which I am planning to do in a subsequent PR), but it is a significant first step in this direction. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 196/64 Mathlib/Algebra/AddConstMap/Equiv.lean,Mathlib/Algebra/Algebra/Equiv.lean,Mathlib/Algebra/Module/Equiv/Basic.lean,Mathlib/Algebra/Module/Equiv/Defs.lean,Mathlib/Algebra/Module/ZLattice/Covolume.lean,Mathlib/Analysis/InnerProductSpace/PiL2.lean,Mathlib/Analysis/InnerProductSpace/TwoDim.lean,Mathlib/Analysis/Normed/Affine/Isometry.lean,Mathlib/Analysis/Normed/Affine/MazurUlam.lean,Mathlib/Analysis/Normed/Operator/Banach.lean,Mathlib/Analysis/Normed/Operator/LinearIsometry.lean,Mathlib/Analysis/NormedSpace/HahnBanach/Extension.lean,Mathlib/GroupTheory/Perm/Option.lean,Mathlib/LinearAlgebra/AffineSpace/AffineEquiv.lean,Mathlib/LinearAlgebra/AffineSpace/ContinuousAffineEquiv.lean,Mathlib/LinearAlgebra/RootSystem/IsValuedIn.lean,Mathlib/Logic/Equiv/Option.lean,Mathlib/MeasureTheory/Measure/Haar/InnerProductSpace.lean,Mathlib/MeasureTheory/Measure/Lebesgue/Complex.lean,Mathlib/ModelTheory/Algebra/Field/IsAlgClosed.lean,Mathlib/NumberTheory/NumberField/Discriminant/Defs.lean,Mathlib/Order/Hom/Basic.lean,Mathlib/Order/Hom/WithTopBot.lean,Mathlib/RingTheory/Bialgebra/Equiv.lean,Mathlib/RingTheory/Coalgebra/Equiv.lean,Mathlib/RingTheory/DedekindDomain/Different.lean,Mathlib/RingTheory/PowerBasis.lean,Mathlib/Topology/Algebra/Module/Equiv.lean,Mathlib/Topology/Algebra/Module/LinearPMap.lean,Mathlib/Topology/MetricSpace/DilationEquiv.lean,Mathlib/Topology/VectorBundle/Basic.lean 31 1 ['github-actions'] nobody
0-83506
23 hours ago
0-83506
23 hours ago
0-84326
23 hours
25190 wwylele
author:wwylele
feat(GroupTheory/Divisible): Add rational SMul and Module This is part of #25140. A torsion-free ℕ-divisible commutative group is a ℚ-module. This new instance could collide with existing instances such as ℚ-module on ℝ that comes from `Algebra`. I don't know how much an issue this is. I set the new instance with low priority so hopefully it won't interfere existing instances. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) awaiting-author 127/0 Mathlib/Data/Rat/Lemmas.lean,Mathlib/GroupTheory/Divisible.lean 2 2 ['eric-wieser', 'github-actions'] nobody
0-76373
21 hours ago
0-76373
21 hours ago
14-31640
14 days
25442 oliver-butterley
author:oliver-butterley
feat(MeasureTheory.VectorMeasure) : add a definition of total variation for VectorMeasure This PR adds variation for any `VectorMeasure` using a supremum definition. Currently mathlib has `TotalVariation` defined for a signed measure using the Hahn-Jordan decomposition, but this doesn't generalise. Includes the result showing that for `SignedMeasure`s the two definitions coincide. Motivation: generally this is an important concept but specifically as a step for proving RMK in the complex case which in turn is a step to prove the spectral theorem. Co-authored-by: @yoh-tanimoto --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) new-contributor RFC 664/0 Mathlib.lean,Mathlib/MeasureTheory/VectorMeasure/Variation.lean 2 4 ['github-actions', 'grunweg', 'oliver-butterley'] nobody
0-37769
10 hours ago
0-38103
10 hours ago
0-38511
10 hours
25230 Thmoas-Guan
author:Thmoas-Guan
feat(Algebra): definition of cohen macaulay In this PR, we added the definition of CM module, CM local ring (extending local ring), and CM ring. We also proved Theorem 30, Chater 6, _Commutative Algebra_, Matsumura. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import 2211/37 Mathlib.lean,Mathlib/Algebra/Category/Grp/Preadditive.lean,Mathlib/Algebra/Homology/ExactSequence.lean,Mathlib/Algebra/Module/Submodule/Lattice.lean,Mathlib/LinearAlgebra/Quotient/Basic.lean,Mathlib/RingTheory/CohenMacaulay/Basic.lean,Mathlib/RingTheory/Ideal/AssociatedPrime/Localization.lean,Mathlib/RingTheory/Ideal/MinimalPrime/Localization.lean,Mathlib/RingTheory/KrullDimension/Module.lean,Mathlib/RingTheory/KrullDimension/Regular.lean,Mathlib/RingTheory/Nakayama.lean,Mathlib/RingTheory/Regular/Category.lean,Mathlib/RingTheory/Regular/Depth.lean,Mathlib/RingTheory/Regular/Ischebeck.lean,Mathlib/RingTheory/Spectrum/Prime/LTSeries.lean,Mathlib/RingTheory/Support.lean 16 n/a ['github-actions', 'leanprover-community-bot-assistant'] nobody
0-25003
6 hours ago
unknown
unknown
25623 mattrobball
author:mattrobball
feat: decidable equality for `Quiver.Path` Given a quiver with decidable equality on its vertices and arrows, we construct an instance of decidable equality for `Quiver.Path`. We proceed through a recursion on the length of the path utilizing an intermediate subtype of uniformly bounded paths `Quiver.Path.BoundedPath`. This was motivated by doing computations on small quivers with Lean. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) 69/0 Mathlib/Combinatorics/Quiver/Path.lean 1 1 ['github-actions'] nobody
0-22514
6 hours ago
0-22603
6 hours ago
0-0
0 seconds
25619 xroblot
author:xroblot
feat(NumberField/CMField): A totally complex abelian extension of ℚ is CM --- - [ ] depends on: #23858 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) blocked-by-other-PR 165/6 Mathlib/Algebra/Field/Subfield/Basic.lean,Mathlib/FieldTheory/Galois/Basic.lean,Mathlib/FieldTheory/IntermediateField/Adjoin/Basic.lean,Mathlib/FieldTheory/IntermediateField/Basic.lean,Mathlib/LinearAlgebra/Dimension/Finrank.lean,Mathlib/NumberTheory/NumberField/CMField.lean,Mathlib/NumberTheory/NumberField/InfinitePlace/Embeddings.lean 7 2 ['github-actions', 'mathlib4-dependent-issues-bot'] nobody
0-19121
5 hours ago
0-35075
9 hours ago
0-118
1 minute
24853 smmercuri
author:smmercuri
feat: dimensions of completions at infinite place extensions Let `L / K` be an extension of number fields. For a fixed `v : InfinitePlace K`, we consider the infinite places `w` of `L` that extend `v`. The main results of this PR are: - `InfinitePlace.sum_ramificationIdx_eq`: the sum over all `w` extending `v` of the ramification indices of `w` over `K` is `[K : L]`. - `InfinitePlace.finrank_eq_ramificationIdx`: the `v.Completion`-dimension of `w.Completion` equals the ramification index of `w` over `K`. --- - [ ] depends on: #24870 - [ ] depends on: #24872 - [ ] depends on: #24873 - [ ] depends on: #24875 - [ ] depends on: #24877 - [x] depends on: #24879 - [ ] depends on: #24881 - [ ] depends on: #24882 - [ ] depends on: #24884 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) large-import FLT merge-conflict blocked-by-other-PR 918/1 Mathlib.lean,Mathlib/Analysis/Normed/Field/WithAbs.lean,Mathlib/Data/Subtype.lean,Mathlib/NumberTheory/NumberField/InfinitePlace/Basic.lean,Mathlib/NumberTheory/NumberField/InfinitePlace/Dimension.lean,Mathlib/NumberTheory/NumberField/InfinitePlace/Embeddings.lean,Mathlib/NumberTheory/NumberField/InfinitePlace/Ramification.lean,Mathlib/Topology/Algebra/UniformRing.lean 8 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
26-16899
26 days ago
26-16901
26 days ago
0-1
1 second
24100 eric-wieser
author:eric-wieser
feat: restore some explicit binders from Lean 3 Part of #24099 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) tech debt merge-conflict awaiting-author 39/42 Mathlib/Data/FinEnum.lean,Mathlib/FieldTheory/Galois/Profinite.lean,Mathlib/Topology/Bases.lean,Mathlib/Topology/Compactness/CompactlyGeneratedSpace.lean,Mathlib/Topology/MetricSpace/IsometricSMul.lean,Mathlib/Topology/Metrizable/CompletelyMetrizable.lean,Mathlib/Topology/Metrizable/Uniformity.lean,Mathlib/Topology/Order.lean,Mathlib/Topology/Order/LowerUpperTopology.lean,Mathlib/Topology/UniformSpace/UniformEmbedding.lean 10 3 ['github-actions', 'grunweg', 'leanprover-community-bot-assistant'] nobody
15-21523
15 days ago
15-21525
15 days ago
34-33204
34 days
24881 smmercuri
author:smmercuri
feat: `InfinitePlace.Extension` API for extensions of infinite places. If `L / K` are fields and `v : InfinitePlace K`, then we define - `v.Extension L` : the subtype of `w : InfinitePlace L` whose restriction to `K` matches `v`. - `isExtension_or_isExtension_conjugate` : if `w` extends `v`, then either `w.embedding` extends `v.embedding` or `conjugate w.embedding` extends `v.embedding` - `IsLift`: class encoding the case where `w` extends `v` and `w.embedding` extends `v.embedding`. - `IsConjugateLift`: class encoding the case where `w` extends `v` and `conjugate w.embedding` extends `v.embedding`. --- - [ ] depends on: #24877 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) merge-conflict blocked-by-other-PR 181/0 Mathlib/NumberTheory/NumberField/InfinitePlace/Embeddings.lean,Mathlib/NumberTheory/NumberField/InfinitePlace/Ramification.lean 2 3 ['github-actions', 'leanprover-community-bot-assistant', 'mathlib4-dependent-issues-bot'] nobody
5-7757
5 days ago
5-7758
5 days ago
0-1074
17 minutes

PRs with contradictory labels

There are currently no PRs with contradictory labels. Congratulations!