src/HOL/Predicate.thy
changeset 36531 19f6e3b0d9b6
parent 36513 70096cbdd4e0
child 37549 a62f742f1d58
--- a/src/HOL/Predicate.thy	Thu Apr 29 15:00:39 2010 +0200
+++ b/src/HOL/Predicate.thy	Thu Apr 29 15:00:40 2010 +0200
@@ -880,10 +880,9 @@
 
 code_abort not_unique
 
-code_reflect
+code_reflect Predicate
   datatypes pred = Seq and seq = Empty | Insert | Join
   functions map
-  module_name Predicate
 
 ML {*
 signature PREDICATE =