Theory BPlusTree_ImpSplitCE
theory BPlusTree_ImpSplitCE
imports
BPlusTree_ImpRange
BPlusTree_ImpSet
BPlusTree_SplitCE
begin
subsection "Obtaining executable code"
text "In order to obtain fully defined functions,
we need to plug our split function implementations
into the locales we introduced previously."
text "Obtaining actual code turns out to be slightly more difficult
due to the use of locales. However, we successfully obtain
the B-tree insertion and membership query with binary search splitting."
global_interpretation bplustree_imp_binary_split_list: split⇩i_list_smeq bin'_split
defines bplustree_isin_list = bplustree_imp_binary_split_list.isin_list⇩i
and bplustree_ins_list = bplustree_imp_binary_split_list.ins_list⇩i
and bplustree_del_list = bplustree_imp_binary_split_list.del_list⇩i
and bplustree_lrange_list = bplustree_imp_binary_split_list.lrange_list⇩i
apply unfold_locales
apply(sep_auto heap: bin'_split_rule)
done
print_theorems