Documentation

Std.Data.DHashMap.AdditionalOperations

Additional dependent hash map operations #

This file defines the operations map and filterMap on Std.Data.DHashMap. We currently do not provide lemmas for these functions.

theorem Std.DHashMap.Raw.WF.filterMap {α : Type u} {β : αType v} {δ : αType w} [BEq α] [Hashable α] {m : Std.DHashMap.Raw α β} (h : m.WF) {f : (a : α) → β aOption (δ a)} :
theorem Std.DHashMap.Raw.WF.map {α : Type u} {β : αType v} {δ : αType w} [BEq α] [Hashable α] {m : Std.DHashMap.Raw α β} (h : m.WF) {f : (a : α) → β aδ a} :
@[inline]
def Std.DHashMap.filterMap {α : Type u} {β : αType v} {δ : αType w} [BEq α] [Hashable α] (f : (a : α) → β aOption (δ a)) (m : Std.DHashMap α β) :

Updates the values of the hash map by applying the given function to all mappings, keeping only those mappings where the function returns some value.

Equations
Instances For
    @[inline]
    def Std.DHashMap.map {α : Type u} {β : αType v} {δ : αType w} [BEq α] [Hashable α] (f : (a : α) → β aδ a) (m : Std.DHashMap α β) :

    Updates the values of the hash map by applying the given function to all mappings.

    Equations
    Instances For