src/HOL/Data_Structures/AA_Map.thy
changeset 68023 75130777ece4
parent 67613 ce654b0e6d69
child 68413 b56ed5010e69
--- a/src/HOL/Data_Structures/AA_Map.thy	Sun Apr 22 21:05:14 2018 +0100
+++ b/src/HOL/Data_Structures/AA_Map.thy	Mon Apr 23 08:09:50 2018 +0200
@@ -23,7 +23,7 @@
      LT \<Rightarrow> adjust (Node lv (delete x l) (a,b) r) |
      GT \<Rightarrow> adjust (Node lv l (a,b) (delete x r)) |
      EQ \<Rightarrow> (if l = Leaf then r
-            else let (l',ab') = del_max l in adjust (Node lv l' ab' r)))"
+            else let (l',ab') = split_max l in adjust (Node lv l' ab' r)))"
 
 
 subsection "Invariance"
@@ -187,7 +187,7 @@
         by(auto simp: post_del_def invar.simps(2))
     next
       assume "l \<noteq> Leaf" thus ?thesis using equal Node.prems
-        by simp (metis inv_l post_del_adjL post_del_max pre_adj_if_postL)
+        by simp (metis inv_l post_del_adjL post_split_max pre_adj_if_postL)
     qed
   qed
 qed (simp add: post_del_def)
@@ -204,7 +204,7 @@
   inorder (delete x t) = del_list x (inorder t)"
 by(induction t)
   (auto simp: del_list_simps inorder_adjust pre_adj_if_postL pre_adj_if_postR 
-              post_del_max post_delete del_maxD split: prod.splits)
+              post_split_max post_delete split_maxD split: prod.splits)
 
 interpretation I: Map_by_Ordered
 where empty = Leaf and lookup = lookup and update = update and delete = delete