theory BPlusTree_Imp imports BPlusTree Partially_Filled_Array Basic_Assn Inst_Ex_Assn begin lemma butlast_double_Cons: "butlast (x#y#xs) = x#(butlast (y#xs))" by auto lemma last_double_Cons: "last (x#y#xs) = (last (y#xs))" by auto section "Imperative B-tree Definition" text "The heap data type definition. Anything stored on the heap always contains data, leafs are represented as None." (* Option as we need a default for non-initializeed entries *)