mathlib4 icon indicating copy to clipboard operation
mathlib4 copied to clipboard

The math library of Lean 4

Results 568 mathlib4 issues
Sort by recently updated
recently updated
newest added

We split `Algebra.Order.Nonneg.Ring` into `Algebra.Order.Nonneg.Ring` which uses unbundled ordered algebra typeclasses, eg `CovariantClass`, and `Algebra.Order.Nonneg.OrderedRing` which uses bundled class, eg `OrderedAddComm`. Using this we can avoid importing bundled ordered algebra...

awaiting-review
merge-conflict
awaiting-CI

--- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/)

WIP

We split `RingTheory.Trace` in `RingTheory.Trace.Defs` and `RingTheory.Trace.Basic`. Similarly for `RingTheory.Norm`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/)

awaiting-review
merge-conflict

In this PR, we set up an instance `SetLike (RingCon R) R` for any `NonUnitalNonAssocRing R`. This enables us to interpret `RingCon R` as two-sided-ideals. Co-authored-by: Eric Wieser --- -...

blocked-by-other-PR
awaiting-review
awaiting-CI
t-algebra

We should be able to use these results about unbundled ordered algebra without importing the heavy machinery of the bundled typeclasses. --- - [ ] depends on: #14393 [![Open in...

blocked-by-other-PR

In this PR, we give a concrete characterization of limit multiforks in the category of types. This contribution was created as part of the AIM workshop "Formalizing algebraic geometry" in...

awaiting-review
t-category-theory
workshop-AIM-AG-2024

Add three elementary lemmas about coefficients of series products. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/)

awaiting-review

--- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/)

WIP
t-algebraic-geometry
workshop-AIM-AG-2024

Thanks Bhavik! --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/)

awaiting-review
easy

The ring theoretic krull dimension is the order theoretic krull dimension applied to its prime spectrum. Unfolding this definition, it is the length of longest series of prime ideals ordered...

awaiting-review
t-algebraic-geometry
t-algebra
new-contributor
workshop-AIM-AG-2024