Skip to content

Commit fd1d6ab

Browse files
committed
more
1 parent 8d61ec3 commit fd1d6ab

File tree

20 files changed

+0
-545
lines changed

20 files changed

+0
-545
lines changed

src/Std/Data/DTreeMap/Basic.lean

Lines changed: 0 additions & 80 deletions
Original file line numberDiff line numberDiff line change
@@ -280,21 +280,13 @@ map is empty.
280280
def minEntry? (t : DTreeMap α β cmp) : Option ((a : α) × β a) :=
281281
letI : Ord α := ⟨cmp⟩; t.inner.minEntry?
282282

283-
@[inline, inherit_doc minEntry?, deprecated minEntry? (since := "2025-03-13")]
284-
def min? (t : DTreeMap α β cmp) : Option ((a : α) × β a) :=
285-
t.minEntry?
286-
287283
/--
288284
Given a proof that the tree map is not empty, retrieves the key-value pair with the smallest key.
289285
-/
290286
@[inline]
291287
def minEntry (t : DTreeMap α β cmp) (h : t.isEmpty = false) : (a : α) × β a :=
292288
letI : Ord α := ⟨cmp⟩; t.inner.minEntry h
293289

294-
@[inline, inherit_doc minEntry, deprecated minEntry (since := "2025-03-13")]
295-
def min (t : DTreeMap α β cmp) (h : t.isEmpty = false) : (a : α) × β a :=
296-
t.minEntry h
297-
298290
/--
299291
Tries to retrieve the key-value pair with the smallest key in the tree map, panicking if the map is
300292
empty.
@@ -303,10 +295,6 @@ empty.
303295
def minEntry! [Inhabited ((a : α) × β a)] (t : DTreeMap α β cmp) : (a : α) × β a :=
304296
letI : Ord α := ⟨cmp⟩; t.inner.minEntry!
305297

306-
@[inline, inherit_doc minEntry!, deprecated minEntry! (since := "2025-03-13")]
307-
def min! [Inhabited ((a : α) × β a)] (t : DTreeMap α β cmp) : (a : α) × β a :=
308-
t.minEntry!
309-
310298
/--
311299
Tries to retrieve the key-value pair with the smallest key in the tree map, returning `fallback` if
312300
the tree map is empty.
@@ -315,10 +303,6 @@ the tree map is empty.
315303
def minEntryD (t : DTreeMap α β cmp) (fallback : (a : α) × β a) : (a : α) × β a :=
316304
letI : Ord α := ⟨cmp⟩; t.inner.minEntryD fallback
317305

318-
@[inline, inherit_doc minEntryD, deprecated minEntryD (since := "2025-03-13")]
319-
def minD (t : DTreeMap α β cmp) (fallback : (a : α) × β a) : (a : α) × β a :=
320-
t.minEntryD fallback
321-
322306
/--
323307
Tries to retrieve the key-value pair with the largest key in the tree map, returning `none` if the
324308
map is empty.
@@ -327,21 +311,13 @@ map is empty.
327311
def maxEntry? (t : DTreeMap α β cmp) : Option ((a : α) × β a) :=
328312
letI : Ord α := ⟨cmp⟩; t.inner.maxEntry?
329313

330-
@[inline, inherit_doc maxEntry?, deprecated maxEntry? (since := "2025-03-13")]
331-
def max? (t : DTreeMap α β cmp) : Option ((a : α) × β a) :=
332-
t.maxEntry?
333-
334314
/--
335315
Given a proof that the tree map is not empty, retrieves the key-value pair with the largest key.
336316
-/
337317
@[inline]
338318
def maxEntry (t : DTreeMap α β cmp) (h : t.isEmpty = false) : (a : α) × β a :=
339319
letI : Ord α := ⟨cmp⟩; t.inner.maxEntry h
340320

341-
@[inline, inherit_doc maxEntry, deprecated maxEntry (since := "2025-03-13")]
342-
def max (t : DTreeMap α β cmp) (h : t.isEmpty = false) : (a : α) × β a :=
343-
t.maxEntry h
344-
345321
/--
346322
Tries to retrieve the key-value pair with the largest key in the tree map, panicking if the map is
347323
empty.
@@ -350,10 +326,6 @@ empty.
350326
def maxEntry! [Inhabited ((a : α) × β a)] (t : DTreeMap α β cmp) : (a : α) × β a :=
351327
letI : Ord α := ⟨cmp⟩; t.inner.maxEntry!
352328

353-
@[inline, inherit_doc maxEntry!, deprecated maxEntry! (since := "2025-03-13")]
354-
def max! [Inhabited ((a : α) × β a)] (t : DTreeMap α β cmp) : (a : α) × β a :=
355-
t.maxEntry!
356-
357329
/--
358330
Tries to retrieve the key-value pair with the largest key in the tree map, returning `fallback` if
359331
the tree map is empty.
@@ -362,10 +334,6 @@ the tree map is empty.
362334
def maxEntryD (t : DTreeMap α β cmp) (fallback : (a : α) × β a) : (a : α) × β a :=
363335
letI : Ord α := ⟨cmp⟩; t.inner.maxEntryD fallback
364336

365-
@[inline, inherit_doc maxEntryD, deprecated maxEntryD (since := "2025-03-13")]
366-
def maxD (t : DTreeMap α β cmp) (fallback : (a : α) × β a) : (a : α) × β a :=
367-
t.maxEntryD fallback
368-
369337
/--
370338
Tries to retrieve the smallest key in the tree map, returning `none` if the map is empty.
371339
-/
@@ -448,37 +416,21 @@ def entryAtIdxD (t : DTreeMap α β cmp) (n : Nat)
448416
def keyAtIdx? (t : DTreeMap α β cmp) (n : Nat) : Option α :=
449417
letI : Ord α := ⟨cmp⟩; Impl.keyAtIdx? t.inner n
450418

451-
@[inline, inherit_doc keyAtIdx?, deprecated keyAtIdx? (since := "2025-03-25")]
452-
def keyAtIndex? (t : DTreeMap α β cmp) (n : Nat) : Option α :=
453-
keyAtIdx? t n
454-
455419
/-- Returns the `n`-th smallest key. -/
456420
@[inline]
457421
def keyAtIdx (t : DTreeMap α β cmp) (n : Nat) (h : n < t.size) : α :=
458422
letI : Ord α := ⟨cmp⟩; Impl.keyAtIdx t.inner t.wf.balanced n h
459423

460-
@[inline, inherit_doc keyAtIdx, deprecated keyAtIdx (since := "2025-03-25")]
461-
def keyAtIndex (t : DTreeMap α β cmp) (n : Nat) (h : n < t.size) : α :=
462-
keyAtIdx t n h
463-
464424
/-- Returns the `n`-th smallest key, or panics if `n` is at least `t.size`. -/
465425
@[inline]
466426
def keyAtIdx! [Inhabited α] (t : DTreeMap α β cmp) (n : Nat) : α :=
467427
letI : Ord α := ⟨cmp⟩; t.inner.keyAtIdx! n
468428

469-
@[inline, inherit_doc keyAtIdx!, deprecated keyAtIdx! (since := "2025-03-25")]
470-
def keyAtIndex! [Inhabited α] (t : DTreeMap α β cmp) (n : Nat) : α :=
471-
keyAtIdx! t n
472-
473429
/-- Returns the `n`-th smallest key, or `fallback` if `n` is at least `t.size`. -/
474430
@[inline]
475431
def keyAtIdxD (t : DTreeMap α β cmp) (n : Nat) (fallback : α) : α :=
476432
letI : Ord α := ⟨cmp⟩; t.inner.keyAtIdxD n fallback
477433

478-
@[inline, inherit_doc keyAtIdxD, deprecated keyAtIdxD (since := "2025-03-25")]
479-
def keyAtIndexD (t : DTreeMap α β cmp) (n : Nat) (fallback : α) : α :=
480-
keyAtIdxD t n fallback
481-
482434
/--
483435
Tries to retrieve the key-value pair with the smallest key that is greater than or equal to the
484436
given key, returning `none` if no such pair exists.
@@ -712,66 +664,34 @@ def getD (t : DTreeMap α β cmp) (a : α) (fallback : β) : β :=
712664
def minEntry? (t : DTreeMap α β cmp) : Option (α × β) :=
713665
letI : Ord α := ⟨cmp⟩; Impl.Const.minEntry? t.inner
714666

715-
@[inline, inherit_doc minEntry?, deprecated minEntry? (since := "2025-03-13")]
716-
def min? (t : DTreeMap α β cmp) : Option (α × β) :=
717-
minEntry? t
718-
719667
@[inline, inherit_doc DTreeMap.minEntry]
720668
def minEntry (t : DTreeMap α β cmp) (h : t.isEmpty = false) : α × β :=
721669
letI : Ord α := ⟨cmp⟩; Impl.Const.minEntry t.inner h
722670

723-
@[inline, inherit_doc minEntry, deprecated minEntry (since := "2025-03-13")]
724-
def min (t : DTreeMap α β cmp) (h : t.isEmpty = false) : α × β :=
725-
minEntry t h
726-
727671
@[inline, inherit_doc DTreeMap.minEntry!]
728672
def minEntry! [Inhabited (α × β)] (t : DTreeMap α β cmp) : α × β :=
729673
letI : Ord α := ⟨cmp⟩; Impl.Const.minEntry! t.inner
730674

731-
@[inline, inherit_doc minEntry!, deprecated minEntry! (since := "2025-03-13")]
732-
def min! [Inhabited (α × β)] (t : DTreeMap α β cmp) : α × β :=
733-
minEntry! t
734-
735675
@[inline, inherit_doc DTreeMap.minEntryD]
736676
def minEntryD (t : DTreeMap α β cmp) (fallback : α × β) : α × β :=
737677
letI : Ord α := ⟨cmp⟩; Impl.Const.minEntryD t.inner fallback
738678

739-
@[inline, inherit_doc minEntryD, deprecated minEntryD (since := "2025-03-13")]
740-
def minD (t : DTreeMap α β cmp) (fallback : α × β) : α × β :=
741-
minEntryD t fallback
742-
743679
@[inline, inherit_doc DTreeMap.maxEntry?]
744680
def maxEntry? (t : DTreeMap α β cmp) : Option (α × β) :=
745681
letI : Ord α := ⟨cmp⟩; Impl.Const.maxEntry? t.inner
746682

747-
@[inline, inherit_doc maxEntry?, deprecated maxEntry? (since := "2025-03-13")]
748-
def max? (t : DTreeMap α β cmp) : Option (α × β) :=
749-
maxEntry? t
750-
751683
@[inline, inherit_doc DTreeMap.maxEntry]
752684
def maxEntry (t : DTreeMap α β cmp) (h : t.isEmpty = false) : α × β :=
753685
letI : Ord α := ⟨cmp⟩; Impl.Const.maxEntry t.inner h
754686

755-
@[inline, inherit_doc maxEntry, deprecated maxEntry (since := "2025-03-13")]
756-
def max (t : DTreeMap α β cmp) (h : t.isEmpty = false) : α × β :=
757-
maxEntry t h
758-
759687
@[inline, inherit_doc DTreeMap.maxEntry!]
760688
def maxEntry! [Inhabited (α × β)] (t : DTreeMap α β cmp) : α × β :=
761689
letI : Ord α := ⟨cmp⟩; Impl.Const.maxEntry! t.inner
762690

763-
@[inline, inherit_doc maxEntry!, deprecated maxEntry! (since := "2025-03-13")]
764-
def max! [Inhabited (α × β)] (t : DTreeMap α β cmp) : α × β :=
765-
maxEntry! t
766-
767691
@[inline, inherit_doc DTreeMap.maxEntryD]
768692
def maxEntryD (t : DTreeMap α β cmp) (fallback : α × β) : α × β :=
769693
letI : Ord α := ⟨cmp⟩; Impl.Const.maxEntryD t.inner fallback
770694

771-
@[inline, inherit_doc maxEntryD, deprecated maxEntryD (since := "2025-03-13")]
772-
def maxD (t : DTreeMap α β cmp) (fallback : α × β) : α × β :=
773-
maxEntryD t fallback
774-
775695
@[inline, inherit_doc DTreeMap.entryAtIdx?]
776696
def entryAtIdx? (t : DTreeMap α β cmp) (n : Nat) : Option (α × β) :=
777697
letI : Ord α := ⟨cmp⟩; Impl.Const.entryAtIdx? t.inner n

src/Std/Data/DTreeMap/Lemmas.lean

Lines changed: 0 additions & 17 deletions
Original file line numberDiff line numberDiff line change
@@ -1297,14 +1297,6 @@ theorem forMUncurried_eq_forM_toList [Monad m] [LawfulMonad m] {f : α × β →
12971297
forMUncurried f t = (Const.toList t).forM f :=
12981298
Impl.Const.forM_eq_forM_toList
12991299

1300-
/--
1301-
Deprecated, use `forMUncurried_eq_forM_toList` together with `forM_eq_forMUncurried` instead.
1302-
-/
1303-
@[deprecated forMUncurried_eq_forM_toList (since := "2025-03-02")]
1304-
theorem forM_eq_forM_toList [Monad m] [LawfulMonad m] {f : α → β → m PUnit} :
1305-
t.forM f = (Const.toList t).forM (fun a => f a.1 a.2) :=
1306-
Impl.Const.forM_eq_forM_toList
1307-
13081300
theorem forIn_eq_forInUncurried [Monad m] [LawfulMonad m]
13091301
{f : α → β → δ → m (ForInStep δ)} {init : δ} :
13101302
t.forIn f init = forInUncurried (fun a b => f a.1 a.2 b) init t := rfl
@@ -1314,15 +1306,6 @@ theorem forInUncurried_eq_forIn_toList [Monad m] [LawfulMonad m]
13141306
forInUncurried f init t = ForIn.forIn (Const.toList t) init f :=
13151307
Impl.Const.forIn_eq_forIn_toList
13161308

1317-
/--
1318-
Deprecated, use `forInUncurried_eq_forIn_toList` together with `forIn_eq_forInUncurried` instead.
1319-
-/
1320-
@[deprecated forInUncurried_eq_forIn_toList (since := "2025-03-02")]
1321-
theorem forIn_eq_forIn_toList [Monad m] [LawfulMonad m]
1322-
{f : α → β → δ → m (ForInStep δ)} {init : δ} :
1323-
t.forIn f init = ForIn.forIn (Const.toList t) init (fun a b => f a.1 a.2 b) :=
1324-
Impl.Const.forIn_eq_forIn_toList
1325-
13261309
end Const
13271310

13281311
end monadic

src/Std/Data/DTreeMap/Raw/Basic.lean

Lines changed: 0 additions & 60 deletions
Original file line numberDiff line numberDiff line change
@@ -202,10 +202,6 @@ def getKeyD (t : Raw α β cmp) (a : α) (fallback : α) : α :=
202202
def minEntry? (t : Raw α β cmp) : Option ((a : α) × β a) :=
203203
letI : Ord α := ⟨cmp⟩; t.inner.minEntry?
204204

205-
@[inline, inherit_doc minEntry?, deprecated minEntry? (since := "2025-03-13")]
206-
def min? (t : Raw α β cmp) : Option ((a : α) × β a) :=
207-
t.minEntry?
208-
209205
/-!
210206
We do not provide `minEntry` for the raw trees.
211207
-/
@@ -214,26 +210,14 @@ We do not provide `minEntry` for the raw trees.
214210
def minEntry! [Inhabited ((a : α) × β a)] (t : Raw α β cmp) : (a : α) × β a :=
215211
letI : Ord α := ⟨cmp⟩; t.inner.minEntry!
216212

217-
@[inline, inherit_doc minEntry!, deprecated minEntry! (since := "2025-03-13")]
218-
def min! [Inhabited ((a : α) × β a)] (t : Raw α β cmp) : (a : α) × β a :=
219-
t.minEntry!
220-
221213
@[inline, inherit_doc DTreeMap.minEntryD]
222214
def minEntryD (t : Raw α β cmp) (fallback : (a : α) × β a) : (a : α) × β a :=
223215
letI : Ord α := ⟨cmp⟩; t.inner.minEntryD fallback
224216

225-
@[inline, inherit_doc minEntryD, deprecated minEntryD (since := "2025-03-13")]
226-
def minD (t : Raw α β cmp) (fallback : (a : α) × β a) : (a : α) × β a :=
227-
t.minEntryD fallback
228-
229217
@[inline, inherit_doc DTreeMap.maxEntry?]
230218
def maxEntry? (t : Raw α β cmp) : Option ((a : α) × β a) :=
231219
letI : Ord α := ⟨cmp⟩; t.inner.maxEntry?
232220

233-
@[inline, inherit_doc maxEntry?, deprecated maxEntry? (since := "2025-03-13")]
234-
def max? (t : Raw α β cmp) : Option ((a : α) × β a) :=
235-
t.maxEntry?
236-
237221
/-!
238222
We do not provide `maxEntry` for the raw trees.
239223
-/
@@ -242,18 +226,10 @@ We do not provide `maxEntry` for the raw trees.
242226
def maxEntry! [Inhabited ((a : α) × β a)] (t : Raw α β cmp) : (a : α) × β a :=
243227
letI : Ord α := ⟨cmp⟩; t.inner.maxEntry!
244228

245-
@[inline, inherit_doc maxEntry!, deprecated maxEntry! (since := "2025-03-13")]
246-
def max! [Inhabited ((a : α) × β a)] (t : Raw α β cmp) : (a : α) × β a :=
247-
t.maxEntry!
248-
249229
@[inline, inherit_doc DTreeMap.maxEntryD]
250230
def maxEntryD (t : Raw α β cmp) (fallback : (a : α) × β a) : (a : α) × β a :=
251231
letI : Ord α := ⟨cmp⟩; t.inner.maxEntryD fallback
252232

253-
@[inline, inherit_doc maxEntryD, deprecated maxEntryD (since := "2025-03-13")]
254-
def maxD (t : Raw α β cmp) (fallback : (a : α) × β a) : (a : α) × β a :=
255-
t.maxEntryD fallback
256-
257233
@[inline, inherit_doc DTreeMap.minKey?]
258234
def minKey? (t : Raw α β cmp) : Option α :=
259235
letI : Ord α := ⟨cmp⟩; t.inner.minKey?
@@ -306,10 +282,6 @@ def entryAtIdxD (t : Raw α β cmp) (n : Nat) (fallback : (a : α) × β a) : (a
306282
def keyAtIdx? (t : Raw α β cmp) (n : Nat) : Option α :=
307283
letI : Ord α := ⟨cmp⟩; Impl.keyAtIdx? t.inner n
308284

309-
@[inline, inherit_doc DTreeMap.keyAtIdx?, deprecated keyAtIdx? (since := "2025-03-25")]
310-
def keyAtIndex? (t : Raw α β cmp) (n : Nat) : Option α :=
311-
keyAtIdx? t n
312-
313285
/-!
314286
We do not provide `keyAtIdx` for the raw trees.
315287
-/
@@ -318,18 +290,10 @@ We do not provide `keyAtIdx` for the raw trees.
318290
def keyAtIdx! [Inhabited α] (t : Raw α β cmp) (n : Nat) : α :=
319291
letI : Ord α := ⟨cmp⟩; t.inner.keyAtIdx! n
320292

321-
@[inline, inherit_doc DTreeMap.keyAtIdx!, deprecated keyAtIdx! (since := "2025-03-25")]
322-
def keyAtIndex! [Inhabited α] (t : Raw α β cmp) (n : Nat) : α :=
323-
keyAtIdx! t n
324-
325293
@[inline, inherit_doc DTreeMap.keyAtIdxD]
326294
def keyAtIdxD (t : Raw α β cmp) (n : Nat) (fallback : α) : α :=
327295
letI : Ord α := ⟨cmp⟩; t.inner.keyAtIdxD n fallback
328296

329-
@[inline, inherit_doc DTreeMap.keyAtIdxD, deprecated keyAtIdxD (since := "2025-03-25")]
330-
def keyAtIndexD (t : Raw α β cmp) (n : Nat) (fallback : α) : α :=
331-
keyAtIdxD t n fallback
332-
333297
@[inline, inherit_doc DTreeMap.getEntryGE?]
334298
def getEntryGE? (t : Raw α β cmp) (k : α) : Option ((a : α) × β a) :=
335299
letI : Ord α := ⟨cmp⟩; Impl.getEntryGE? k t.inner
@@ -464,10 +428,6 @@ def getD (t : Raw α β cmp) (a : α) (fallback : β) : β :=
464428
def minEntry? (t : Raw α β cmp) : Option (α × β) :=
465429
letI : Ord α := ⟨cmp⟩; Impl.Const.minEntry? t.inner
466430

467-
@[inline, inherit_doc minEntry?, deprecated minEntry? (since := "2025-03-13")]
468-
def min? (t : Raw α β cmp) : Option (α × β) :=
469-
minEntry? t
470-
471431
/-!
472432
We do not provide `minEntry` for the raw trees.
473433
-/
@@ -476,42 +436,22 @@ We do not provide `minEntry` for the raw trees.
476436
def minEntry! [Inhabited (α × β)] (t : Raw α β cmp) : α × β :=
477437
letI : Ord α := ⟨cmp⟩; Impl.Const.minEntry! t.inner
478438

479-
@[inline, inherit_doc minEntry!, deprecated minEntry! (since := "2025-03-13")]
480-
def min! [Inhabited (α × β)] (t : Raw α β cmp) : α × β :=
481-
minEntry! t
482-
483439
@[inline, inherit_doc DTreeMap.Const.minEntryD]
484440
def minEntryD (t : Raw α β cmp) (fallback : α × β) : α × β :=
485441
letI : Ord α := ⟨cmp⟩; Impl.Const.minEntryD t.inner fallback
486442

487-
@[inline, inherit_doc minEntryD, deprecated minEntryD (since := "2025-03-13")]
488-
def minD (t : Raw α β cmp) (fallback : α × β) : α × β :=
489-
minEntryD t fallback
490-
491443
@[inline, inherit_doc DTreeMap.Const.maxEntry?]
492444
def maxEntry? (t : Raw α β cmp) : Option (α × β) :=
493445
letI : Ord α := ⟨cmp⟩; Impl.Const.maxEntry? t.inner
494446

495-
@[inline, inherit_doc maxEntry?, deprecated maxEntry? (since := "2025-03-13")]
496-
def max? (t : Raw α β cmp) : Option (α × β) :=
497-
maxEntry? t
498-
499447
@[inline, inherit_doc DTreeMap.Const.maxEntry!]
500448
def maxEntry! [Inhabited (α × β)] (t : Raw α β cmp) : α × β :=
501449
letI : Ord α := ⟨cmp⟩; Impl.Const.maxEntry! t.inner
502450

503-
@[inline, inherit_doc maxEntry!, deprecated maxEntry! (since := "2025-03-13")]
504-
def max! [Inhabited (α × β)] (t : Raw α β cmp) : α × β :=
505-
maxEntry! t
506-
507451
@[inline, inherit_doc DTreeMap.Const.maxEntryD]
508452
def maxEntryD (t : Raw α β cmp) (fallback : α × β) : α × β :=
509453
letI : Ord α := ⟨cmp⟩; Impl.Const.maxEntryD t.inner fallback
510454

511-
@[inline, inherit_doc maxEntryD, deprecated maxEntryD (since := "2025-03-13")]
512-
def maxD (t : Raw α β cmp) (fallback : α × β) : α × β :=
513-
maxEntryD t fallback
514-
515455
@[inline, inherit_doc DTreeMap.Const.entryAtIdx?]
516456
def entryAtIdx? (t : Raw α β cmp) (n : Nat) : Option (α × β) :=
517457
letI : Ord α := ⟨cmp⟩; Impl.Const.entryAtIdx? t.inner n

src/Std/Data/DTreeMap/Raw/Lemmas.lean

Lines changed: 0 additions & 26 deletions
Original file line numberDiff line numberDiff line change
@@ -1305,32 +1305,6 @@ theorem forMUncurried_eq_forM_toList [Monad m] [LawfulMonad m] {f : α × β →
13051305
forMUncurried f t = (Const.toList t).forM f :=
13061306
Impl.Const.forM_eq_forM_toList
13071307

1308-
/--
1309-
Deprecated, use `forMUncurried_eq_forM_toList` together with `forM_eq_forMUncurried` instead.
1310-
-/
1311-
@[deprecated forMUncurried_eq_forM_toList (since := "2025-03-02")]
1312-
theorem forM_eq_forM_toList [Monad m] [LawfulMonad m] {f : α → β → m PUnit} :
1313-
t.forM f = (Const.toList t).forM (fun a => f a.1 a.2) :=
1314-
Impl.Const.forM_eq_forM_toList
1315-
1316-
theorem forIn_eq_forInUncurried [Monad m] [LawfulMonad m]
1317-
{f : α → β → δ → m (ForInStep δ)} {init : δ} :
1318-
t.forIn f init = forInUncurried (fun a b => f a.1 a.2 b) init t := rfl
1319-
1320-
theorem forInUncurried_eq_forIn_toList [Monad m] [LawfulMonad m]
1321-
{f : α × β → δ → m (ForInStep δ)} {init : δ} :
1322-
forInUncurried f init t = ForIn.forIn (Const.toList t) init f :=
1323-
Impl.Const.forIn_eq_forIn_toList
1324-
1325-
/--
1326-
Deprecated, use `forInUncurried_eq_forIn_toList` together with `forIn_eq_forInUncurried` instead.
1327-
-/
1328-
@[deprecated forInUncurried_eq_forIn_toList (since := "2025-03-02")]
1329-
theorem forIn_eq_forIn_toList [Monad m] [LawfulMonad m]
1330-
{f : α → β → δ → m (ForInStep δ)} {init : δ} :
1331-
t.forIn f init = ForIn.forIn (Const.toList t) init (fun a b => f a.1 a.2 b) :=
1332-
Impl.Const.forIn_eq_forIn_toList
1333-
13341308
end Const
13351309

13361310
end monadic

0 commit comments

Comments
 (0)