Documentation

Std.Data.DTreeMap.Raw.Iterator

Iterators on DTreeMap.Raw #

@[inline]
def Std.DTreeMap.Raw.iter {α : Type u} {β : αType v} {cmp : ααOrdering} (m : Raw α β cmp) :
Iter ((a : α) × β a)

Returns a finite iterator over the entries of a dependent tree map. The iterator yields the elements of the map in order and then terminates.

Termination properties:

  • Finite instance: always
  • Productive instance: always
Equations
Instances For
    @[inline]
    def Std.DTreeMap.Raw.keysIter {α : Type u} {β : αType u} {cmp : ααOrdering} (m : Raw α β cmp) :
    Iter α

    Returns a finite iterator over the keys of a dependent tree map. The iterator yields the keys in order and then terminates.

    The key and value types must live in the same universe.

    Termination properties:

    • Finite instance: always
    • Productive instance: always
    Equations
    Instances For
      @[inline]
      def Std.DTreeMap.Raw.valuesIter {α β : Type u} {cmp : ααOrdering} (m : Raw α (fun (x : α) => β) cmp) :
      Iter β

      Returns a finite iterator over the values of a tree map. The iterator yields the values in order and then terminates.

      The key and value types must live in the same universe.

      Termination properties:

      • Finite instance: always
      • Productive instance: always
      Equations
      Instances For
        @[simp]
        theorem Std.DTreeMap.Raw.toList_iter {α : Type u_1} {β : αType u_2} {cmp : ααOrdering} (m : Raw α β cmp) :
        @[simp]
        theorem Std.DTreeMap.Raw.keysIter_toList {α : Type u_1} {β : αType u_1} {cmp : ααOrdering} (m : Raw α β cmp) :
        @[simp]
        theorem Std.DTreeMap.Raw.valuesIter_toList {α β : Type u_1} {cmp : ααOrdering} (m : Raw α (fun (x : α) => β) cmp) :