Documentation

Std.Data.Iterators.Producers.Monadic.Empty

This file provides an empty iterator.

structure Std.Iterators.Empty (m : Type w → Type w') (β : Type w) :

The internal state of the IterM.empty iterator.

    Instances For
      @[inline]
      def Std.Iterators.IterM.empty (m : Type w → Type w') (β : Type w) :
      IterM m β

      Returns an iterator that terminates immediately.

      Termination properties:

      • Finite instance: always
      • Productive instance: always
      Equations
      Instances For
        def Std.Iterators.Empty.PlausibleStep {m : Type w → Type w'} {β : Type w} :
        IterM m β(step : IterStep (IterM m β) β) → Prop
        Equations
        Instances For
          instance Std.Iterators.Empty.instIterator {m : Type w → Type w'} {β : Type w} [Monad m] :
          Iterator (Empty m β) m β
          Equations
          instance Std.Iterators.Empty.instFinite {m : Type w → Type w'} {β : Type w} [Monad m] :
          Finite (Empty m β) m