Documentation

Std.Data.DHashMap.Internal.List.Sublist

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: tiny private implementation of List.Sublist

inductive Std.DHashMap.Internal.List.Sublist {α : Type u} :
List αList αProp

Internal implementation detail of the hash map

Instances For
    theorem Std.DHashMap.Internal.List.Sublist.length_le {α : Type u} {l₁ : List α} {l₂ : List α} (h : Std.DHashMap.Internal.List.Sublist l₁ l₂) :
    l₁.length l₂.length
    @[simp]
    theorem Std.DHashMap.Internal.List.Sublist.cons_iff {α : Type u} {a : α} {l₁ : List α} {l₂ : List α} :
    theorem Std.DHashMap.Internal.List.Sublist.map {α : Type u} {β : Type v} (f : αβ) {l₁ : List α} {l₂ : List α} (h : Std.DHashMap.Internal.List.Sublist l₁ l₂) :
    theorem Std.DHashMap.Internal.List.Sublist.mem {α : Type u} {l₁ : List α} {l₂ : List α} (h : Std.DHashMap.Internal.List.Sublist l₁ l₂) {a : α} :
    a l₁a l₂