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

These lemmas are separate from the rest and need not be pulled in by the main file.

awaiting-review
merge-conflict

- [x] Depends on: #735 - [x] Depends on: #737 - [x] Depends on: #738 This adds RBMap lemmas corresponding to all of the RBSet lemmas.

awaiting-review
merge-conflict

I also added some lemmas in List.Lemmas that were necessary. I'm not sure about the naming of some of the lemmas I added, so I would appreciate feedback!

awaiting-review
merge-conflict

```Lean4 theorem forall_mem_iff_forall_index [DecidableEq α] {p : α → Prop} {l : List α} : (∀ x ∈ l, p x) ↔ (∀ i : Fin (l.length), p (l.get i))...

awaiting-author
merge-conflict

This caught 14 bugs with no false positives over in https://github.com/leanprover-community/mathlib4/pull/10899

awaiting-author
merge-conflict

`List.insertP` is a generalized, tail-recursive version of the insert step in insertion-sort. Sample use: ```lean def insertionSort [LT α] [DecidableRel (α:=α) (· < ·)] (l : List α) := l.foldl...

awaiting-review

This is a tactic that allows targeted unfolding of expressions in the proof state by specifying patterns and occurrences (an idea that is due to Yaël Dillies). The file `Utils.lean`...

awaiting-author
merge-conflict

I've made a new version of Lean's `DiscrTree` called `RefinedDiscrTree` with a lot of new features. It is able to index lambda's, forall's, and their bound variables. It also gives...

awaiting-author
merge-conflict

This proof has three different hypotheses named `h`, and in a upcoming version of leanprover/lean4#2793 something is going to change in how they shadow each other. This is a fix...

depends on core changes
merge-conflict

awaiting-author
merge-conflict