src/HOL/Data_Structures/RBT_Set.thy
changeset 68440 6826718f732d
parent 68431 b294e095f64c
child 68998 818898556504
equal deleted inserted replaced
68439:c8101022e52a 68440:6826718f732d
   254 theorem rbt_delete: "rbt t \<Longrightarrow> rbt (delete k t)"
   254 theorem rbt_delete: "rbt t \<Longrightarrow> rbt (delete k t)"
   255 by (metis delete_def rbt_def color_paint_Black del_invc_invh invc_paint_Black invc2I invh_paint)
   255 by (metis delete_def rbt_def color_paint_Black del_invc_invh invc_paint_Black invc2I invh_paint)
   256 
   256 
   257 text \<open>Overall correctness:\<close>
   257 text \<open>Overall correctness:\<close>
   258 
   258 
   259 interpretation Set_by_Ordered
   259 interpretation S: Set_by_Ordered
   260 where empty = empty and isin = isin and insert = insert and delete = delete
   260 where empty = empty and isin = isin and insert = insert and delete = delete
   261 and inorder = inorder and inv = rbt
   261 and inorder = inorder and inv = rbt
   262 proof (standard, goal_cases)
   262 proof (standard, goal_cases)
   263   case 1 show ?case by (simp add: empty_def)
   263   case 1 show ?case by (simp add: empty_def)
   264 next
   264 next