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

Change the behavior of the infoview to visually distinguish: * frozen instances * typeclass assumptions that are not instances * unfrozen typeclass assumptions * non typeclass assumptions --- The style...

RFC
awaiting-review

Define * `seminormed_group` * `seminormed_add_group` * `seminormed_comm_group` * `normed_group` * `normed_add_group` * `normed_comm_group` Additivize all lemmas in `analysis.normed.group.basic`. To disambiguate names, I add one or two `'` to the multiplicative...

awaiting-review
t-analysis

This PR constructs a linear order on `finsupp`s where both source and target are linearly ordered. This is useful for #15983, where these linear orders are used to prove that...

awaiting-review
t-order

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

awaiting-author
delegated
t-algebra

Restate lemmas using `monoid_with_zero_hom_class`/`ring_hom_class` instead of `monoid_with_zero_hom`/`ring_hom`. --- - [ ] depends on: #15985 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/)

awaiting-review
blocked-by-other-PR
awaiting-CI

Define `pfun.prod : (α →. γ) → (β →. δ) → α × β →. γ × δ`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/)

awaiting-review

From LTE Author: Johan Commelin [Zulip discussion](https://leanprover.zulipchat.com/#narrow/stream/267928-condensed-mathematics/topic/extremally.20disconnected.20sets) --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/)

WIP
awaiting-author

to match `smul_comm_class` and `vadd_assoc_class`. --- [Zulip](https://leanprover.zulipchat.com/#narrow/stream/116395-maths/topic/left.20vs.20right.20modules.20in.20tensor.20products/near/261974400), [other Zulip](https://leanprover.zulipchat.com/#narrow/stream/113488-general/topic/smul_assoc_class) [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/)

awaiting-review

Fix the linting errors coming from `fintype_finite`, `to_additive_doc` and `doc_blame`. Pull out a `[projective_plane P L]` assumption to a `variables` declaration in `combinatorics.configuration`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/)

awaiting-review

This PR proves that the lexicographic linear order on finitely supported functions preserves (one) covariant class assumption. This is a further step in proving that many `add_monoid_algebra`s have no zero-divisors....

blocked-by-other-PR
t-order