src/HOL/Finite_Set.thy
changeset 37767 a2b7a20d6ea3
parent 37678 0040bafffdef
child 37770 cddb3106adb8
--- a/src/HOL/Finite_Set.thy	Mon Jul 12 08:58:27 2010 +0200
+++ b/src/HOL/Finite_Set.thy	Mon Jul 12 10:48:37 2010 +0200
@@ -589,7 +589,7 @@
 inductive_cases empty_fold_graphE [elim!]: "fold_graph f z {} x"
 
 definition fold :: "('a \<Rightarrow> 'b \<Rightarrow> 'b) \<Rightarrow> 'b \<Rightarrow> 'a set \<Rightarrow> 'b" where
-[code del]: "fold f z A = (THE y. fold_graph f z A y)"
+  "fold f z A = (THE y. fold_graph f z A y)"
 
 text{*A tempting alternative for the definiens is
 @{term "if finite A then THE y. fold_graph f z A y else e"}.