batteries icon indicating copy to clipboard operation
batteries copied to clipboard

The "batteries included" extended library for the Lean programming language and theorem prover

Results 164 batteries issues
Sort by recently updated
recently updated
newest added

Note this includes the parallelisation upgrade that is still being reviewed at Mathlib as https://github.com/leanprover-community/mathlib4/pull/8435, but Leo is keen to get this into Std so I'm opening this already. Depends...

help wanted
depends on another PR
merge-conflict

This powers up `solve_by_elim` by allowing it to use projections of hypotheses. It does so by saturating the context with let-bindings for projections (recursively). For interactive use of `solve_by_elim`, this...

awaiting-review
merge-conflict

Mathlib has `.docker` and `.devcontainer` folders that (for one thing) make it easy to quickly load in to a fresh install of lean + mathlib (eg with gitpod.io). I think...

Also move `Std.Logic` to `Std.Logic.Basic`.

awaiting-author
merge-conflict

Integrates a few of Mathlib's lemmas over `List`s. Some proofs have been slightly simplified

awaiting-review
merge-conflict

``` import Std /---/ def npowRec {M : Type} [Mul M] (one : M) : Nat → M → M | 0, _ => one | n + 1, a...

I feel like this might already exist somewhere, but with a not too old Std/Mathlib imported it does not exist yet.

awaiting-author
merge-conflict

awaiting-review
merge-conflict

this goes along https://github.com/leanprover/lean4/pull/2577

WIP
depends on core changes
merge-conflict