Documentation

Std.Data.DHashMap.Internal.List.HashesTo

This is an internal implementation file of the hash map. Users of the hash map should not rely on the contents of this file.

File contents: lemmas about HashesTo (defined in Internal.Defs)

@[simp]
theorem Std.DHashMap.Internal.List.hashesTo_nil {α : Type u} {β : αType v} [BEq α] [Hashable α] {i : Nat} {size : Nat} :
theorem Std.DHashMap.Internal.List.hashesTo_cons {α : Type u} {β : αType v} [BEq α] [Hashable α] {i : Nat} {size : Nat} {l : List ((a : α) × β a)} {k : α} {v : β k} (h : ∀ (h' : 0 < size), (Std.DHashMap.Internal.mkIdx size h' (hash k)).val.toNat = i) :
theorem Std.DHashMap.Internal.List.HashesTo.containsKey_eq_false {α : Type u} {β : αType v} [BEq α] [Hashable α] [LawfulHashable α] {l : List ((a : α) × β a)} {i : Nat} {size : Nat} (hs : 0 < size) (h : Std.DHashMap.Internal.List.HashesTo l i size) (k : α) :