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

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

awaiting-review
easy

also move `lTensor_inj_iff_rTensor_inj` to `LinearMap` --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/)

awaiting-review
t-algebra
maintainer-merge

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

awaiting-review
t-algebra

In this PR, we define `lipschitzGroup`, `pinGroup` and `spinGroup`, and prove some basic lemmas. Ported from leanprover-community/mathlib/pull/16040. Co-authored-by: Jiale Miao Co-authored-by: Eric Wieser --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/) This PR is...

awaiting-author
new-contributor

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

awaiting-review
t-algebra

--- - [ ] depends on: #12434 [part one: submodule version] - [x] depends on: #11635 - [x] depends on: #11598 [need `finsuppTensorFinsupp'_symm_single`] - [x] depends on: #11731 - [x]...

WIP
blocked-by-other-PR
t-algebra

Order/SuccPred/Basic.lean: add `SuccOrder.ofLinearWellFoundedLT`, which puts a SuccOrder on an arbitrary well-ordered type. Also add the dual, `PredOrder` version. Add missing `pred` lemmas corresponding to existing `succ` lemmas. Order/SuccPred/Limit.lean: add `SuccOrder.limitRecOn`...

delegated
t-order
t-logic

Define cocountable and cocardinal filters. Any feedback on the way these are phrased and written is more than welcome! --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/)

awaiting-author
merge-conflict
t-topology
t-order

A construction by transfinite recursion, fairly standard in set theory, but I have yet to see similar arguments in mathlib. See [module docstring](https://github.com/leanprover-community/mathlib4/blob/Field_Card_Emb/Mathlib/SetTheory/Cardinal/FieldEmb.lean#L20-L137) for more details. I use some ad...

t-algebra
t-logic

1. if $A$ is a noetherian graded ring, then $A_0$ is a noetherian subring of $A$ and $A$ is a finitely generated algebra over $A_0$, if $M$ is a finitely...

WIP
merge-conflict