batteries
batteries copied to clipboard
The "batteries included" extended library for the Lean programming language and theorem prover
It was still present in the namespaces `Std.Tactic.Lint` and `Std.CodeAction`.
This is to correct a name clash from #528 with Mathlib pointed out by @eric-wieser We add `List.finRange` and `Array.finRange` (with basic lemmas). The synonyms `Fin.list` and `Fin.enum` are deprecated.
These have been recently requested on [Zulip](https://leanprover.zulipchat.com/#narrow/stream/270676-lean4/topic/Regarding.20map.20and.20extract.20for.20Byte.2FFloatArrays/near/452971124).
Alternative to #836. While this is not quite a drop-in replacement for users of Mathlib's `ByteSlice`, it offers the same functionality while using the same basic structure as core's `Subarray`...
These were previously moved to core (verbatim) in leanprover/lean4#3290.