diff -r 374caac3d624 -r 3e11f35496b3 src/HOL/Data_Structures/Set2_Join_RBT.thy --- a/src/HOL/Data_Structures/Set2_Join_RBT.thy Sun Sep 15 17:24:31 2019 +0200 +++ b/src/HOL/Data_Structures/Set2_Join_RBT.thy Mon Sep 16 18:00:27 2019 +0200 @@ -101,7 +101,7 @@ (* unused *) lemma rbt_join: "\ invc l; invh l; invc r; invh r \ \ rbt(join l x r)" -by(simp add: invc2_joinL invc2_joinR invc_paint_Black invh_joinL invh_joinR invh_paint rbt_def +by(simp add: invc2_joinL invc2_joinR invh_joinL invh_joinR invh_paint rbt_def color_paint_Black join_def) text \To make sure the the black height is not increased unnecessarily:\ @@ -206,7 +206,7 @@ by(auto simp: bst_paint bst_joinL bst_joinR join_def) lemma inv_join: "\ invc l; invh l; invc r; invh r \ \ invc(join l x r) \ invh(join l x r)" -by (simp add: invc2_joinL invc2_joinR invc_paint_Black invh_joinL invh_joinR invh_paint join_def) +by (simp add: invc2_joinL invc2_joinR invh_joinL invh_joinR invh_paint join_def) subsubsection "Interpretation of \<^locale>\Set2_Join\ with Red-Black Tree"