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

Let R be a Dedekind domain with field of fractions K. This PR does two things: 1) makes the finite adeles of K/R into a K-algebra 2) turns `finiteAdeleRing` into...

awaiting-author
t-number-theory
t-algebra

In additive combinatorics, a pretty standard tool called Chang's lemma uses a version of linear independence and linear span with "scalars" restricted to `{-1, 0, 1}`. This PR defines those...

awaiting-review
merge-conflict
t-combinatorics

Add version of `ker_liftQ_eq_bot` with both-ways `≤` replaced by `=` in the hypotheses. --- Because of proof irrelevance, the `le_of_eq h` in the goal doesn't really matter. It'll unify with...

awaiting-review
t-algebra

Equivalence between the quotient by a binary sum of submodules and an iterated quotient. --- This is a very useful "rewrite rule" when doing algebra, especially if you're doing some...

awaiting-review
t-algebra

These instances make it possible to argue with multiplication and inequalities in `ℤₘ₀` . --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) These instances are in a bit of a funny place (they need...

awaiting-review
t-algebra

Move the material about `Invertible` to files under `Algebra.Group`, `Algebra.GroupWithZero`, `Algebra.Ring`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/)

ready-to-merge
t-algebra
maintainer-merge
move-decls

Move its lemmas (mostly) to two new files: * `Algebra.Order.Group.Basic` for the lemmas about group-like objects * `Algebra.Order.Ring.Basic` for the lemmas about ring-like objects --- - [ ] depends on:...

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

Introduces the category `ContAction V G` for any concrete category `V` with a forgetful functor to `TopCat` and monoid `G`. It is realized as a full subcategory of `Action V...

ready-to-merge
t-category-theory

In this category, we shall show that if `C` is a monoidal category and `W` is a class of morphism that is preserved by the tensor product, then the localized...

WIP
t-category-theory

Unlike the Python version, this script also supports set_option tactics and terms, and we add a couple of tests. --- Mentored by @digama0; thanks for all your help. Written at...

awaiting-review
t-linter
tech debt