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:
Finiteinstance: alwaysProductiveinstance: 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:
Finiteinstance: alwaysProductiveinstance: always
Equations
- m.keysIter = Std.Iterators.Iter.map (fun (e : (a : α) × β a) => e.fst) m.iter
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:
Finiteinstance: alwaysProductiveinstance: always
Equations
- m.valuesIter = Std.Iterators.Iter.map (fun (e : (_ : α) × β) => e.snd) m.iter
Instances For
@[simp]
theorem
Std.DTreeMap.Raw.valuesIter_toList
{α β : Type u_1}
{cmp : α → α → Ordering}
(m : Raw α (fun (x : α) => β) cmp)
: