mathlib4
mathlib4 copied to clipboard
The math library of Lean 4
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...
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...
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...
--- - [ ] depends on: #14429 [](https://gitpod.io/from-referrer/)
--- [](https://gitpod.io/from-referrer/)
--- [](https://gitpod.io/from-referrer/)
We add `PowerBasis.exists_sModEq`. From `flt-regular`. --- [](https://gitpod.io/from-referrer/)
--- [](https://gitpod.io/from-referrer/)
```lean theorem mem_rec_on {C : Seq α → Prop} {a s} (M : a ∈ s) (h1 : ∀ b s', a = b ∨ C s' → C (cons...
--- [](https://gitpod.io/from-referrer/)