Theory Pairing_Heap.Pairing_Heap_List1
section ‹Pairing Heap According to Okasaki›
theory Pairing_Heap_List1
imports
"HOL-Library.Multiset"
"HOL-Library.Pattern_Aliases"
"HOL-Data_Structures.Priority_Queue_Specs"
begin
subsection ‹Definitions›
text
‹This implementation follows Okasaki \<^cite>‹"Okasaki"›.
It satisfies the invariant that ‹Empty› only occurs
at the root of a pairing heap. The functional correctness proof does not
require the invariant but the amortized analysis (elsewhere) makes use of it.›