Skip to content

Commit 2d2ad36

Browse files
fgdoraisleanprover-community-mathlib4-botlinesthatinterlace
committed
chore: adaptations for batteries#1491 (#31334)
After [batteries#1491](leanprover-community/batteries#1491) is merged: - [x] Edit the lakefile to point to leanprover-community/batteries:main - [x] Run lake update batteries - [x] Merge leanprover-community/mathlib4:master - [ ] Wait for CI and merge Co-authored-by: leanprover-community-mathlib4-bot <leanprover-community-mathlib4-bot@users.noreply.github.com> Co-authored-by: F. G. Dorais <fgdorais@gmail.com> Co-authored-by: Wrenna Robson <wrenna.robson@bristol.ac.uk>
1 parent c6b3276 commit 2d2ad36

File tree

2 files changed

+1
-9
lines changed

2 files changed

+1
-9
lines changed

Mathlib/Data/List/Sublists.lean

Lines changed: 0 additions & 8 deletions
Original file line numberDiff line numberDiff line change
@@ -118,14 +118,6 @@ theorem sublistsAux_eq_flatMap :
118118
rw [flatMap_append, ← ih, flatMap_singleton, sublistsAux, foldl_append]
119119
simp [sublistsAux])
120120

121-
@[csimp] theorem sublists_eq_sublistsFast : @sublists = @sublistsFast := by
122-
ext α l : 2
123-
trans l.foldr sublistsAux [[]]
124-
· rw [sublistsAux_eq_flatMap, sublists]
125-
· simp only [sublistsFast, sublistsAux_eq_array_foldl]
126-
rw [← foldr_hom Array.toList]
127-
· intros; congr
128-
129121
theorem sublists_append (l₁ l₂ : List α) :
130122
sublists (l₁ ++ l₂) = (sublists l₂) >>= (fun x => (sublists l₁).map (· ++ x)) := by
131123
simp only [sublists, foldr_append]

lake-manifest.json

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -65,7 +65,7 @@
6565
"type": "git",
6666
"subDir": null,
6767
"scope": "leanprover-community",
68-
"rev": "dd3edb3aa6b4de87f96f2c3998881ef95ba24ed7",
68+
"rev": "02402d27841c9b46ca2d69d344c94b3ed022fee2",
6969
"name": "batteries",
7070
"manifestFile": "lake-manifest.json",
7171
"inputRev": "main",

0 commit comments

Comments
 (0)