src/HOL/ex/Execute_Choice.thy
changeset 64267 b9a1486e79be
parent 61933 cf58b5b794b2
child 66453 cc19f7ca2ed6
--- a/src/HOL/ex/Execute_Choice.thy	Sun Oct 16 22:43:51 2016 +0200
+++ b/src/HOL/ex/Execute_Choice.thy	Mon Oct 17 11:46:22 2016 +0200
@@ -54,7 +54,7 @@
   "finite (Mapping.keys M) \<Longrightarrow> x \<in> Mapping.keys M \<Longrightarrow> y \<in> Mapping.keys M \<Longrightarrow>
     the (Mapping.lookup M x) + valuesum (Mapping.delete x M) =
     the (Mapping.lookup M y) + valuesum (Mapping.delete y M)"
-  unfolding valuesum_def  by transfer (simp add: setsum_diff)
+  unfolding valuesum_def  by transfer (simp add: sum_diff)
 
 text \<open>
   Given \<open>valuesum_rec\<close> as initial description, we stepwise refine it to something executable;