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

It turns out that pushing the dependency out is quite annoying, so as an alternative, we propose considering Preorder, PartialOrder and LinearOrder to be foundational type classes that all of...

awaiting-author
merge-conflict
maintainer-merge

Adds a `MorphismProperty.stalkwise` constructor for morphism properties of schemes from a property of ring homomorphisms. Also adds API for reducing proofs of stability under base change to affine situations for...

awaiting-review
merge-conflict
t-algebraic-geometry

Follows up on Yael's comment in #8612 by making `n` (in `x ^ (p ^ n)`) explicit. --- - [ ] depends on: #8612 Lucas' Theorem CI should fail in...

blocked-by-other-PR
new-contributor

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

WIP
blocked-by-other-PR
awaiting-CI
t-algebraic-geometry

--- [![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/)

WIP

We add `PowerBasis.exists_sModEq`. From `flt-regular`. --- [![Open in Gitpod](https://gitpod.io/button/open-in-gitpod.svg)](https://gitpod.io/from-referrer/)

awaiting-review
t-algebra

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

WIP

```lean theorem mem_rec_on {C : Seq α → Prop} {a s} (M : a ∈ s) (h1 : ∀ b s', a = b ∨ C s' → C (cons...

WIP
blocked-by-other-PR

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

awaiting-review
t-analysis