simplified BLAST_DATA;
authorwenzelm
Sat, 14 May 2011 13:32:33 +0200
changeset 42802 51d7e74f6899
parent 42801 da4ad5f98953
child 42803 7ed59879b1b6
simplified BLAST_DATA;
src/FOL/FOL.thy
src/HOL/HOL.thy
src/Provers/blast.ML
--- a/src/FOL/FOL.thy	Sat May 14 13:26:55 2011 +0200
+++ b/src/FOL/FOL.thy	Sat May 14 13:32:33 2011 +0200
@@ -201,7 +201,7 @@
   structure Blast = Blast
   (
     structure Classical = Cla
-    val thy = @{theory}
+    val Trueprop_const = dest_Const @{const Trueprop}
     val equality_name = @{const_name eq}
     val not_name = @{const_name Not}
     val notE = @{thm notE}
--- 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}
--- a/src/Provers/blast.ML	Sat May 14 13:26:55 2011 +0200
+++ b/src/Provers/blast.ML	Sat May 14 13:32:33 2011 +0200
@@ -41,7 +41,7 @@
 signature BLAST_DATA =
 sig
   structure Classical: CLASSICAL
-  val thy: theory
+  val Trueprop_const: string * typ
   val equality_name: string
   val not_name: string
   val notE: thm           (* [| ~P;  P |] ==> R *)
@@ -172,8 +172,7 @@
 fun isGoal (Const ("*Goal*", _) $ _) = true
   | isGoal _ = false;
 
-val TruepropC = Object_Logic.judgment_name Data.thy;  (* FIXME *)
-val TruepropT = Sign.the_const_type Data.thy TruepropC;
+val (TruepropC, TruepropT) = Data.Trueprop_const;
 
 fun mk_Trueprop t = Term.$ (Term.Const (TruepropC, TruepropT), t);