adapted to new implicit claset mechanism;
authorwenzelm
Mon, 03 Nov 1997 11:56:17 +0100
changeset 4078 c107ab1c7626
parent 4077 8ce7c713968c
child 4079 9df5e4f22d96
adapted to new implicit claset mechanism;
src/Provers/blast.ML
--- a/src/Provers/blast.ML	Mon Nov 03 11:48:56 1997 +0100
+++ b/src/Provers/blast.ML	Mon Nov 03 11:56:17 1997 +0100
@@ -1,4 +1,4 @@
-(*  Title: 	Provers/blast
+(*  Title: 	Provers/blast.ML
     ID:         $Id$
     Author: 	Lawrence C Paulson, Cambridge University Computer Laboratory
     Copyright   1997  University of Cambridge
@@ -60,7 +60,7 @@
   val contr_tac 	: int -> tactic
   val dup_intr		: thm -> thm
   val vars_gen_hyp_subst_tac : bool -> int -> tactic
-  val claset		: claset ref
+  val claset		: unit -> claset
   val rep_claset	: 
       claset -> {safeIs: thm list, safeEs: thm list, 
 		 hazIs: thm list, hazEs: thm list,
@@ -1165,7 +1165,7 @@
 
 fun blast_tac cs = (DEEPEN (1,20) (depth_tac cs) 0);
 
-fun Blast_tac i = blast_tac (!Data.claset) i;
+fun Blast_tac i = blast_tac (Data.claset()) i;
 
 
 (*** For debugging: these apply the prover to a subgoal and return 
@@ -1184,7 +1184,7 @@
      end
      handle Subscript => error("There is no subgoal " ^ Int.toString i));
 
-fun Trygl lim i = trygl (!Data.claset) lim i;
+fun Trygl lim i = trygl (Data.claset()) lim i;
 
 (*Read a string to make an initial, singleton branch*)
 fun readGoal sign s = read_cterm sign (s,propT) |>
@@ -1193,7 +1193,7 @@
 fun tryInThy thy lim s = 
     (fullTrace:=[];  trail := [];  ntrail := 0;
      timeap prove (sign_of thy, 
-		   !Data.claset, 
+		   Data.claset(), 
 		   [initBranch ([readGoal (sign_of thy) s], lim)], 
 		   I));