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
trafficstars

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

awaiting-review
easy

The classes `BoundedSub` and `BoundedMul` were added in PRs #12559 and #12790 to generalize subtraction and multiplication operations on bounded continuous functions (especially for the case of codomain `NNReal`). The...

WIP
t-topology
t-analysis

https://leanprover.zulipchat.com/#narrow/stream/270676-lean4/topic/cc.20tactic.20comes.20to.20Lean4 --- - [x] depends on: #11960 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/)

awaiting-review
modifies-tactic-syntax
mathlib-port
t-meta

Move the basic content of `GroupTheory.GroupAction` to new folders `Algebra.Group.Action` and `Algebra.GroupWithZero.Action` depending on whether it is additivisable or not. --- - [x] depends on: #12974 - [x] depends on:...

awaiting-review
merge-conflict
awaiting-CI
RFC
t-algebra

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

merge-conflict
new-contributor

--- Split out from #12937 (suggestions there applied here) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/)

awaiting-review
t-algebra

This PR defines the following equiv: ```lean def Ideal.associatesNonZeroDivisorsEquivIsPrincipal : Associates R⁰ ≃ {I : (Ideal R)⁰ // IsPrincipal (I : Ideal R)} ``` Also, move the definition `Ideal.associatesEquivIsPrincipal` from...

blocked-by-other-PR
awaiting-author
t-algebra

Prove that `{0, ..., k - 1} ⊆ ℤ/(n + 1)ℤ` and `{0, ..., k - 1} ⊆ ℕ` are `m`-Freiman isomorphic if `m * k ≤ n` --- -...

awaiting-review
t-combinatorics

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

WIP
blocked-by-other-PR
merge-conflict
t-number-theory

This is consistent with the `Group` file, and drops the dependency on `Mathlib.Order` entirely. --- - [x] depends on: #13008 - [x] depends on: #13033 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/)

awaiting-review
merge-conflict
move-decls