mathlib icon indicating copy to clipboard operation
mathlib copied to clipboard

Lean 3's obsolete mathematical components library: please use mathlib4

Results 381 mathlib issues
Sort by recently updated
recently updated
newest added

--- - [x] depends on: #13963 I wasn't able to redefine `game` as `antisymmetrization pgame (≤)`. For whatever reason, that broke a few instances of the `⟦x⟧` notation. [![Open in...

WIP
awaiting-CI
too-late

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

WIP
too-late

The `recommend` tactic searches for lemmas in the current environment that look like they could be useful to prove the current goal. It is based on premise selection heuristic used...

t-meta
modifies-tactic-syntax
not-too-late

Define the Jacobson radical of a ring as the intersection of all maximal left ideals, and prove basic properties: famous equivalent conditions for an element in a ring to be...

awaiting-author
too-late

* Add `codisjoint.inf_left_sup_inf_right` and `is_compl.le_inf_sup_inf`. * Add `filter.comap_ite`, `filter.comap_max`, and `filter.tendsto_ite`. * Add `real.map_to_nnreal_at_top`, `real.comap_to_nnreal_at_top`, and `real.tendsto_to_nnreal_at_top_iff`. * Rename `tendsto_real_to_nnreal` to `filter.tendsto.real_to_nnreal` so that it can be used with dot...

awaiting-author
t-topology
t-order
modifies-synchronized-file
too-late

This is another tracking issue for me, but if anyone is interested in helping out, then I would be very happy. The goal is to get tempered distributions and the...

long term
t-analysis

Basic arithmetic of quadratic fields (ring of integers, discriminant and so on) should now not be too difficult. [https://en.wikipedia.org/wiki/Quadratic_field](https://en.wikipedia.org/wiki/Quadratic_field) [https://en.wikipedia.org/wiki/Quadratic_integer](https://en.wikipedia.org/wiki/Quadratic_integer)

feature-request

As part of the porting process to Lean 4, we should refactor mathlib to remove occurences of ```lean local attribute [semireducible] foobar attribute [irreducible] xyzzy ``` The following data is...

needs-refactor
mathport

Prior to #18163, the behavior was to sort based on the repr, meaning, that `{0, 5, 10}` is sorted as `{0, 10, 5}`. After #18163, the order is non-deterministic and...

* [x] Define Banach algebras: it turns out that we already have `normed_algebra`s; * [ ] Prove facts about convergence of series for Banach algebras; * [ ] Migrate some...

feature-request