@@ -512,7 +512,7 @@ where finally
512512 refine ⟨1 , ?_⟩
513513 simpa [succMany?_one] using hs
514514
515- private theorem Iterator.instIteratorLoop.loop_eq_loopWf [UpwardEnumerable α] [LE α] [DecidableLE α]
515+ private theorem Iterator.instIteratorLoop.loop_eq_wf [UpwardEnumerable α] [LE α] [DecidableLE α]
516516 [LawfulUpwardEnumerable α] [LawfulUpwardEnumerableLE α] [Monad n] [LawfulMonad n]
517517 {γ LargeEnough hl upperBound} {next hn} {acc} (Pl wf f) :
518518 loop γ LargeEnough hl upperBound acc next hn (fun out h₁ h₂ acc => Subtype.val <$> f out h₁ h₂ acc) =
@@ -620,7 +620,7 @@ instance Iterator.instLawfulIteratorLoop [UpwardEnumerable α] [LE α] [Decidabl
620620 split; rotate_left
621621 · simp [Monadic.step_eq_step, Monadic.step, Internal.LawfulMonadLiftBindFunction.liftBind_pure]
622622 rename_i next _
623- rw [instIteratorLoop.loop_eq_loopWf Pl wf, instIteratorLoop.loopWf_eq (lift := lift)]
623+ rw [instIteratorLoop.loop_eq_wf Pl wf, instIteratorLoop.loopWf_eq (lift := lift)]
624624 simp only [Monadic.step_eq_step, Monadic.step, instLawfulMonadLiftFunction.liftBind_pure,
625625 Shrink.inflate_deflate]
626626 split
@@ -1110,7 +1110,7 @@ where finally
11101110 refine ⟨1 , ?_⟩
11111111 simpa [succMany?_one] using hs
11121112
1113- private theorem Iterator.instIteratorLoop.loop_eq_loopWf [UpwardEnumerable α] [LT α] [DecidableLT α]
1113+ private theorem Iterator.instIteratorLoop.loop_eq_wf [UpwardEnumerable α] [LT α] [DecidableLT α]
11141114 [LawfulUpwardEnumerable α] [LawfulUpwardEnumerableLT α] [Monad n] [LawfulMonad n]
11151115 {γ LargeEnough hl upperBound} {next hn} {acc} (Pl wf f) :
11161116 loop γ LargeEnough hl upperBound acc next hn (fun out h₁ h₂ acc => Subtype.val <$> f out h₁ h₂ acc) =
@@ -1218,7 +1218,7 @@ instance Iterator.instLawfulIteratorLoop [UpwardEnumerable α] [LT α] [Decidabl
12181218 split; rotate_left
12191219 · simp [Monadic.step_eq_step, Monadic.step, Internal.LawfulMonadLiftBindFunction.liftBind_pure]
12201220 rename_i next _
1221- rw [instIteratorLoop.loop_eq_loopWf Pl wf, instIteratorLoop.loopWf_eq (lift := lift)]
1221+ rw [instIteratorLoop.loop_eq_wf Pl wf, instIteratorLoop.loopWf_eq (lift := lift)]
12221222 simp only [Monadic.step_eq_step, Monadic.step, instLawfulMonadLiftFunction.liftBind_pure,
12231223 Shrink.inflate_deflate]
12241224 split
@@ -1614,7 +1614,7 @@ where finally
16141614 refine ⟨1 , ?_⟩
16151615 simpa [succMany?_one] using hs
16161616
1617- private theorem Iterator.instIteratorLoop.loop_eq_loopWf [UpwardEnumerable α]
1617+ private theorem Iterator.instIteratorLoop.loop_eq_wf [UpwardEnumerable α]
16181618 [LawfulUpwardEnumerable α] [Monad n] [LawfulMonad n]
16191619 {γ LargeEnough hl} {next hn} {acc} (Pl wf f) :
16201620 loop γ LargeEnough hl acc next hn (fun out h acc => Subtype.val <$> f out h acc) =
@@ -1707,7 +1707,7 @@ instance Iterator.instLawfulIteratorLoop [UpwardEnumerable α]
17071707 split; rotate_left
17081708 · simp [Monadic.step_eq_step, Monadic.step, Internal.LawfulMonadLiftBindFunction.liftBind_pure]
17091709 rename_i next _
1710- rw [instIteratorLoop.loop_eq_loopWf Pl wf, instIteratorLoop.loopWf_eq (lift := lift)]
1710+ rw [instIteratorLoop.loop_eq_wf Pl wf, instIteratorLoop.loopWf_eq (lift := lift)]
17111711 simp only [Monadic.step_eq_step, Monadic.step, instLawfulMonadLiftFunction.liftBind_pure,
17121712 Shrink.inflate_deflate]
17131713 apply bind_congr; intro forInStep
0 commit comments