src/HOL/Predicate.thy
changeset 37767 a2b7a20d6ea3
parent 37549 a62f742f1d58
child 38651 8aadda8e1338
--- a/src/HOL/Predicate.thy	Mon Jul 12 08:58:27 2010 +0200
+++ b/src/HOL/Predicate.thy	Mon Jul 12 10:48:37 2010 +0200
@@ -408,10 +408,10 @@
   "P \<squnion> Q = Pred (eval P \<squnion> eval Q)"
 
 definition
-  [code del]: "\<Sqinter>A = Pred (INFI A eval)"
+  "\<Sqinter>A = Pred (INFI A eval)"
 
 definition
-  [code del]: "\<Squnion>A = Pred (SUPR A eval)"
+  "\<Squnion>A = Pred (SUPR A eval)"
 
 definition
   "- P = Pred (- eval P)"
@@ -873,7 +873,7 @@
 
 definition the :: "'a pred => 'a"
 where
-  [code del]: "the A = (THE x. eval A x)"
+  "the A = (THE x. eval A x)"
 
 lemma the_eq[code]: "the A = singleton (\<lambda>x. not_unique A) A"
 by (auto simp add: the_def singleton_def not_unique_def)