src/HOL/ex/Execute_Choice.thy
changeset 39198 f967a16dfcdd
parent 37595 9591362629e3
child 39302 d7728f65b353
--- a/src/HOL/ex/Execute_Choice.thy	Mon Sep 06 22:58:06 2010 +0200
+++ b/src/HOL/ex/Execute_Choice.thy	Tue Sep 07 10:05:19 2010 +0200
@@ -26,7 +26,7 @@
   case True then show ?thesis by (simp add: is_empty_def keys_def valuesum_def)
 next
   case False
-  then have l: "\<exists>l. l \<in> dom (Mapping.lookup m)" by (auto simp add: is_empty_def expand_fun_eq mem_def keys_def)
+  then have l: "\<exists>l. l \<in> dom (Mapping.lookup m)" by (auto simp add: is_empty_def ext_iff mem_def keys_def)
   then have "(let l = SOME l. l \<in> dom (Mapping.lookup m) in
      the (Mapping.lookup m l) + (\<Sum>k \<in> dom (Mapping.lookup m) - {l}. the (Mapping.lookup m k))) =
        (\<Sum>k \<in> dom (Mapping.lookup m). the (Mapping.lookup m k))"