batteries
batteries copied to clipboard
The "batteries included" extended library for the Lean programming language and theorem prover
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...
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...
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`.
Integrates a few of Mathlib's lemmas over `List`s. Some proofs have been slightly simplified
``` 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.
this goes along https://github.com/leanprover/lean4/pull/2577