Skip to content

Commit d0e5669

Browse files
committed
chore: bump Std to #253 (#7113)
Bump PR for leanprover-community/batteries#253 Co-authored-by: Scott Morrison <scott.morrison@gmail.com>
1 parent 6de5329 commit d0e5669

File tree

2 files changed

+2
-9
lines changed

2 files changed

+2
-9
lines changed

Mathlib/Control/Basic.lean

Lines changed: 1 addition & 8 deletions
Original file line numberDiff line numberDiff line change
@@ -6,6 +6,7 @@ Authors: Johannes Hölzl
66
import Mathlib.Init.Control.Combinators
77
import Mathlib.Tactic.CasesM
88
import Mathlib.Tactic.Attr.Core
9+
import Std.Data.List.Basic
910

1011
#align_import control.basic from "leanprover-community/mathlib"@"48fb5b5280e7c81672afc9524185ae994553ebf4"
1112

@@ -77,14 +78,6 @@ variable {m : Type u → Type v} [Monad m] [LawfulMonad m]
7778

7879
open List
7980

80-
/-- A generalization of `List.partition` which partitions the list according to a monadic
81-
predicate. `List.partition` corresponds to the case where `f = Id`. -/
82-
def List.partitionM {f : TypeType} [Monad f] {α : Type} (p : α → f Bool) :
83-
List α → f (List α × List α)
84-
| [] => pure ([], [])
85-
| x :: xs => condM (p x)
86-
(Prod.map (cons x) id <$> List.partitionM p xs)
87-
(Prod.map id (cons x) <$> List.partitionM p xs)
8881
#align list.mpartition List.partitionM
8982

9083
theorem map_bind (x : m α) {g : α → m β} {f : β → γ} :

lake-manifest.json

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -36,7 +36,7 @@
3636
{"git":
3737
{"url": "https://github.com/leanprover/std4",
3838
"subDir?": null,
39-
"rev": "e8c27f7d90ee71470558efd1bc197fe55068c748",
39+
"rev": "2a10db96d0ea1c00d0b30d2bbcea7e7b4584ffba",
4040
"opts": {},
4141
"name": "std",
4242
"inputRev?": "main",

0 commit comments

Comments
 (0)