batteries
                                
                                
                                
                                    batteries copied to clipboard
                            
                            
                            
                        The "batteries included" extended library for the Lean programming language and theorem prover
`String.splitOn_of_valid` is the first of the eleven unproved theorems about strings. I added the following to prove it: * lemmas about `Nat.add` and lists * the file `Batteries.Data.List.SplitOnList` * the...
`List.isEmpty_iff_eq_nil` and `List.modifyHead_modifyHead` are from `Mathlib.Data.List.Basic`. We need these theorems to prove `String.splitOn_of_valid`. See https://github.com/leanprover-community/batteries/pull/743. Batteries bump PR in Mathlib: https://github.com/leanprover-community/mathlib4/pull/12540 Co-authored-by: Kim Morrison --- - [x] depends-on: https://github.com/leanprover-community/batteries/pull/790
This is an attempt to switch to using `lake test`. Gradually more of this functionality will be taken over by `lake`, but I would like to push this along and...
- [x] Depends on: #735 - [x] Depends on: #737 - [x] Depends on: #738 This adds `RBSet.upperBound?` symmetric to `lowerBound?`, and lifts all the RBNode theorems to RBSet (and...
Quick fix for #770.
This adds an implementation of exact (IEEE conforming) rounding from `Rat` to `Float` rounding nearest ties to even. Note that unlike most other lean functions (but like most float functions),...