src/HOL/HOL.thy
changeset 33364 2bd12592c5e8
parent 33316 6a72af4e84b8
child 33369 470a7b233ee5
--- a/src/HOL/HOL.thy	Fri Oct 30 14:02:42 2009 +0100
+++ b/src/HOL/HOL.thy	Fri Oct 30 18:32:40 2009 +0100
@@ -1818,7 +1818,7 @@
 
 code_datatype "TYPE('a\<Colon>{})"
 
-code_datatype Trueprop "prop"
+code_datatype "prop" Trueprop
 
 text {* Code equations *}