Documentation

Std.Data.Iterators.Lemmas.Producers.Empty

@[simp]
@[simp]
theorem Std.Iterators.Iter.forIn_empty {m : Type u_1 → Type u_2} {β γ : Type u_1} [Monad m] [LawfulMonad m] {init : γ} {f : βγm (ForInStep γ)} :
forIn (empty β) init f = pure init
@[simp]
theorem Std.Iterators.Iter.foldM_empty {m : Type u_1 → Type u_2} {β γ : Type u_1} [Monad m] [LawfulMonad m] {init : γ} {f : γβm γ} :
foldM f init (empty β) = pure init
@[simp]
theorem Std.Iterators.Iter.fold_empty {β γ : Type u_1} {init : γ} {f : γβγ} :
fold f init (empty β) = init