Theory MapStdImpl

Up to index of Isabelle/HOL/Collections

theory MapStdImpl
imports ListMapImpl_Invar HashMap TrieMapImpl ArrayHashMap ArrayMapImpl
(*  Title:       Isabelle Collections Library
Author: Peter Lammich <peter dot lammich at uni-muenster.de>
Maintainer: Peter Lammich <peter dot lammich at uni-muenster.de>
*)

header "Standard Implementations of Maps"
theory MapStdImpl
imports
ListMapImpl ListMapImpl_Invar RBTMapImpl HashMap TrieMapImpl ArrayHashMap
ArrayMapImpl
begin
text_raw {*\label{thy:MapStdImpl}*}
text {*
This theory summarizes various standard implementation of maps, namely list-maps, RB-tree-maps, trie-maps, hashmaps, indexed array maps.
*}

end