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 is definition "computes better", so it is needed when showing `from_Spec` and `to_Spec` are inverses - [x] depends on: #16693 --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/)

awaiting-author

* A subgroup has index two if and only if there exists `a` such that for all `b`, `b * a ∈ H` is equivalent to `b ∉ H`. *...

awaiting-author
t-algebra

If $A, B$ are abelian categories and $L\dashv R$ is a pair of adjoint functors, where $L$ is faithful and exact, then enough invectiveness of $B$ implies that of $A$...

awaiting-author
awaiting-CI
t-category-theory

This proof felt a bit painful - I suspect most of the results I needed already exist somewhere else. This `decomposition` instances inherits the noncomputability of `orthogonal_projection`, but it is...

awaiting-author

`nat.divisors` unconditionally preserves multiplication, so this bundles it as a monoid hom, similar for `nat.divisors_antidiagonal`. This PR also changes `nat.divisors` to be defined in terms of `nat.divisors_antidiagonal`, which drastically simplifies...

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

Benefits: - The tactic is faster - The tactic is easier to port to Lean 4 Downside: - The tactic doesn't do any heavy-lifting for the user Zulip thread: https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/wlog/near/296996966...

ready-to-merge
please-adopt
t-meta
delegated
modifies-tactic-syntax

This PR adds: - Group instance for `π_(n+1)` - Commutative group instance for `π_(n+2)` --- - [x] depends on: #16879 [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/)

WIP

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

awaiting-review
t-algebra
t-order

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

awaiting-review
merge-conflict
t-analysis