src/HOL/Library/Enum.thy
changeset 37765 26bdfb7b680b
parent 37678 0040bafffdef
child 38857 97775f3e8722
--- a/src/HOL/Library/Enum.thy	Mon Jul 12 08:58:12 2010 +0200
+++ b/src/HOL/Library/Enum.thy	Mon Jul 12 08:58:13 2010 +0200
@@ -149,7 +149,7 @@
 begin
 
 definition
-  [code del]: "enum = map (\<lambda>ys. the o map_of (zip (enum\<Colon>'a list) ys)) (n_lists (length (enum\<Colon>'a\<Colon>enum list)) enum)"
+  "enum = map (\<lambda>ys. the o map_of (zip (enum\<Colon>'a list) ys)) (n_lists (length (enum\<Colon>'a\<Colon>enum list)) enum)"
 
 instance proof
   show "UNIV = set (enum \<Colon> ('a \<Rightarrow> 'b) list)"
@@ -278,7 +278,7 @@
 begin
 
 definition
-  [code del]: "enum = map (split Char) (product enum enum)"
+  "enum = map (split Char) (product enum enum)"
 
 lemma enum_chars [code]:
   "enum = chars"