src/Pure/search.ML
changeset 15531 08c8dad8e399
parent 14160 6750ff1dfc32
child 15570 8d8c70b41bab
--- a/src/Pure/search.ML	Fri Feb 11 18:51:00 2005 +0100
+++ b/src/Pure/search.ML	Sun Feb 13 17:15:14 2005 +0100
@@ -58,13 +58,13 @@
   Suppresses duplicate solutions to minimize search space.*)
 fun DEPTH_FIRST satp tac = 
  let val tac = tracify trace_DEPTH_FIRST tac
-     fun depth used [] = None
+     fun depth used [] = NONE
        | depth used (q::qs) =
 	  case Seq.pull q of
-	      None         => depth used qs
-	    | Some(st,stq) => 
+	      NONE         => depth used qs
+	    | SOME(st,stq) => 
 		if satp st andalso not (gen_mem eq_thm (st, used))
-		then Some(st, Seq.make
+		then SOME(st, Seq.make
 			         (fn()=> depth (st::used) (stq::qs)))
 		else depth used (tac st :: stq :: qs)
   in  traced_tac (fn st => depth [] ([Seq.single st]))  end;
@@ -156,10 +156,10 @@
 			     implode (map (fn _ => "*") qs))
 		else ();
 		Seq.pull q) of
-	     None         => depth (bnd,inc) qs
-	   | Some(st,stq) => 
+	     NONE         => depth (bnd,inc) qs
+	   | SOME(st,stq) => 
 	       if satp st	(*solution!*)
-	       then Some(st, Seq.make
+	       then SOME(st, Seq.make
 			 (fn()=> depth (bnd,inc) ((k,np,rgd,stq)::qs)))
 
 	       else 
@@ -197,8 +197,8 @@
 val trace_BEST_FIRST = ref false;
 
 (*For creating output sequence*)
-fun some_of_list []     = None
-  | some_of_list (x::l) = Some (x, Seq.make (fn () => some_of_list l));
+fun some_of_list []     = NONE
+  | some_of_list (x::l) = SOME (x, Seq.make (fn () => some_of_list l));
 
 (*Check for and delete duplicate proof states*)
 fun deleteAllMin prf heap = 
@@ -219,7 +219,7 @@
 					(map pairsize nonsats, nprf_heap)) 
 	      | (sats,_)  => some_of_list sats)
       and next nprf_heap =
-            if ThmHeap.is_empty nprf_heap then None
+            if ThmHeap.is_empty nprf_heap then NONE
 	    else 
 	    let val (n,prf) = ThmHeap.min nprf_heap
 	    in if !trace_BEST_FIRST 
@@ -266,8 +266,8 @@
               else (l,m,th)::(l',n,th')::nths;
 
 (*For creating output sequence*)
-fun some_of_list []     = None
-  | some_of_list (x::l) = Some (x, Seq.make (fn () => some_of_list l));
+fun some_of_list []     = NONE
+  | some_of_list (x::l) = SOME (x, Seq.make (fn () => some_of_list l));
 
 val trace_ASTAR = ref false; 
 
@@ -280,7 +280,7 @@
 		 => next (foldr insert_with_level (map cost nonsats, nprfs))
           | (sats,_)  => some_of_list sats)
       end and    
-      next []  = None
+      next []  = NONE
         | next ((level,n,prf)::nprfs)  =
             (if !trace_ASTAR 
                then tracing("level = " ^ string_of_int level ^