Documentation

Std.Data.HashMap.AdditionalOperations

Additional hash map operations #

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

theorem Std.HashMap.Raw.WF.filterMap {α : Type u} {β : Type v} {γ : Type w} [BEq α] [Hashable α] {m : Std.HashMap.Raw α β} {f : αβOption γ} (h : m.WF) :
theorem Std.HashMap.Raw.WF.map {α : Type u} {β : Type v} {γ : Type w} [BEq α] [Hashable α] {m : Std.HashMap.Raw α β} {f : αβγ} (h : m.WF) :
@[inline]
def Std.HashMap.filterMap {α : Type u} {β : Type v} {γ : Type w} [BEq α] [Hashable α] (f : αβOption γ) (m : Std.HashMap α β) :

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.HashMap.map {α : Type u} {β : Type v} {γ : Type w} [BEq α] [Hashable α] (f : αβγ) (m : Std.HashMap α β) :

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

    Equations
    Instances For