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

In the `Monoid` instances for `Function.End α`, `Equiv.Perm α`, `Monoid.End α`, `AddMonoid.End α`, `α →+* α`, replace the default `npowRec` by a custom one in terms of `Nat.iterate`. Write the...

awaiting-review
t-algebra

This PR introduces a structure containing the data involved in a fully faithful functor `F`, i.e. inverse maps to `F.map`. (This was suggested by Andrew Yang.) This should also restore...

awaiting-review
t-category-theory

The bug fix lean4#4206 causes some change in the behaviour of `congr`, `convert` and friends. So some proofs need to be fixed, usually by providing more arguments. --- [![Open in...

merge-conflict
new-contributor

Also used the new simp lemmas to golf `AlgebraicGeometry/ProjectiveSpectrum/*` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/)

awaiting-review
t-algebraic-geometry

Move all the declarations using the mathlib order hierarchy to a new file `Order.Fin`. There were a bunch of order embeddings in `Data.Fin.Basic`, so I kept an embedding version of...

awaiting-review
merge-conflict
t-order

--- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) The working branch for this project is [greedoid-defs](https://github.com/leanprover-community/mathlib4/tree/greedoid-defs). This branch does not contain all features of the working branch, and is for real contribution to Mathlib....

awaiting-review
t-combinatorics

The `subsingleton` tactic tries to close equality goals by arguing that the underlying type is a subsingleton type. It might be via a `Subsingleton` instance (via `Subsingleton.elim`), but it also...

awaiting-review
t-meta

This file seems to frequently confuse `WithBot.some` and `Option.some`, and some of the lemmas are strange as a result. By teaching `cases` not to introduce `Option.some`, we no longer need...

define `rieszContentAux` under `Λ : C(X, ℝ) →ₗ[ℝ] ℝ) (hΛ : ∀ (f : C(X, ℝ)), 0 ≤ f → 0 ≤ Λ f)` and prove that it is a...

WIP
awaiting-review
RFC
t-measure-probability
new-contributor

Adds some lemmas about the coefficient of polynomials of the form `X s ^ n`. Upstreamed from another project. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/)

awaiting-review
t-algebra