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

This PR adds `root_set_prod` (based on `roots_prod`) and cleans up lemma statements (the file already has `{R S : Type*} [field R]`). --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/)

awaiting-review
t-algebra

This PR proves that if `p` splits in a field extensions, then adjoining all of the roots of `p` gives a splitting field of `p`. --- - [x] depends on:...

awaiting-review
t-algebra

We add some documentation, and golf slightly by marking `nat.elim` and `nat.cases` as `reducible`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/)

awaiting-author

iterated_deriv.lean was not used anywhere, and derivative.lean already had independent variants of several of the lemmas there, without the `iterated_deriv` indirecion. It seems better to consolidate these results. --- I...

awaiting-review

Define Heyting-regular elements of an Heyting lattice, namely those `a` such that `aᶜᶜ = a`, and prove that they form a boolean algebra. --- - [ ] depends on: #15305...

awaiting-review
blocked-by-other-PR

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

awaiting-review

Define (generalized) Heyting, co-Heyting and bi-Heyting algebras. --- - [x] depends on: #15302 - [x] depends on: #15304 - [x] depends on: #15340 This a second go at #5527. I...

awaiting-review

introduce H-spaces and prove basic properties, in particular that every topological group is a H-space and that the path space at a point is a H-space. --- - depends on:...

awaiting-review
t-topology

Fix the linting errors coming from `fintype_finite`, `to_additive_doc` and `doc_blame`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/)

awaiting-review

`⌊f a⌋ = ⌊a⌋`, `⌈f a⌉ = ⌈a⌉` and similar for `f` a strictly monotone ring homomorphism. --- - [ ] depends on: #16024 @eric-wieser, those are the lemmas I...

awaiting-review
blocked-by-other-PR