src/HOL/Library/RBT_Impl.thy
changeset 62390 842917225d56
parent 62093 bd73a2279fcd
child 63040 eb4ddd18d635
equal deleted inserted replaced
62380:29800666e526 62390:842917225d56
   153 proof (induct t)
   153 proof (induct t)
   154   case Empty then show ?case by simp
   154   case Empty then show ?case by simp
   155 next
   155 next
   156   case (Branch color t1 a b t2)
   156   case (Branch color t1 a b t2)
   157   let ?A = "Set.insert a (dom (rbt_lookup t1) \<union> dom (rbt_lookup t2))"
   157   let ?A = "Set.insert a (dom (rbt_lookup t1) \<union> dom (rbt_lookup t2))"
   158   have "dom (rbt_lookup (Branch color t1 a b t2)) \<subseteq> ?A" by (auto split: split_if_asm)
   158   have "dom (rbt_lookup (Branch color t1 a b t2)) \<subseteq> ?A" by (auto split: if_split_asm)
   159   moreover from Branch have "finite (insert a (dom (rbt_lookup t1) \<union> dom (rbt_lookup t2)))" by simp
   159   moreover from Branch have "finite (insert a (dom (rbt_lookup t1) \<union> dom (rbt_lookup t2)))" by simp
   160   ultimately show ?case by (rule finite_subset)
   160   ultimately show ?case by (rule finite_subset)
   161 qed 
   161 qed 
   162 
   162 
   163 end
   163 end