src/HOL/HOL.thy
changeset 42802 51d7e74f6899
parent 42799 4e33894aec6d
child 43560 d1650e3720fd
--- a/src/HOL/HOL.thy	Sat May 14 13:26:55 2011 +0200
+++ b/src/HOL/HOL.thy	Sat May 14 13:32:33 2011 +0200
@@ -929,7 +929,7 @@
   structure Blast = Blast
   (
     structure Classical = Classical
-    val thy = @{theory}
+    val Trueprop_const = dest_Const @{const Trueprop}
     val equality_name = @{const_name HOL.eq}
     val not_name = @{const_name Not}
     val notE = @{thm notE}