src/HOL/Mutabelle/mutabelle_extra.ML
changeset 42361 23f352990944
parent 42179 24662b614fd4
child 42429 7691cc61720a
child 42435 c3d880b13aa9
--- a/src/HOL/Mutabelle/mutabelle_extra.ML	Sat Apr 16 15:47:52 2011 +0200
+++ b/src/HOL/Mutabelle/mutabelle_extra.ML	Sat Apr 16 16:15:37 2011 +0200
@@ -122,7 +122,7 @@
   TimeLimit.timeLimit (seconds (!Auto_Tools.time_limit))
       (fn _ =>
           let
-            val [result] = Quickcheck.test_goal_terms (change_options (ProofContext.init_global thy))
+            val [result] = Quickcheck.test_goal_terms (change_options (Proof_Context.init_global thy))
               (false, false) [] [(t, [])]
           in
             case Quickcheck.counterexample_of result of 
@@ -139,7 +139,7 @@
  
 fun invoke_solve_direct thy t =
   let
-    val state = Proof.theorem NONE (K I) (map (single o rpair []) [t]) (ProofContext.init_global thy) 
+    val state = Proof.theorem NONE (K I) (map (single o rpair []) [t]) (Proof_Context.init_global thy) 
   in
     case Solve_Direct.solve_direct false state of
       (true, _) => (Solved, [])
@@ -152,7 +152,7 @@
 
 fun invoke_try thy t =
   let
-    val state = Proof.theorem NONE (K I) (map (single o rpair []) [t]) (ProofContext.init_global thy)
+    val state = Proof.theorem NONE (K I) (map (single o rpair []) [t]) (Proof_Context.init_global thy)
   in
     case Try.invoke_try (SOME (seconds 5.0)) ([], [], [], []) state of
       true => (Solved, [])
@@ -196,7 +196,7 @@
 
 fun invoke_nitpick thy t =
   let
-    val ctxt = ProofContext.init_global thy
+    val ctxt = Proof_Context.init_global thy
     val state = Proof.init ctxt
     val (res, _) = Nitpick.pick_nits_in_term state
       (Nitpick_Isar.default_params thy []) false 1 1 1 [] [] t
@@ -312,7 +312,7 @@
 
 fun is_executable_term thy t =
   let
-    val ctxt = ProofContext.init_global thy
+    val ctxt = Proof_Context.init_global thy
   in
     can (TimeLimit.timeLimit (seconds 2.0)
       (Quickcheck.test_goal_terms
@@ -414,7 +414,7 @@
 (*          |> filter (not o is_forbidden_mutant) *)
           |> List.mapPartial (try (Sign.cert_term thy))
           |> List.filter (is_some o try (Thm.cterm_of thy))
-          |> List.filter (is_some o try (Syntax.check_term (ProofContext.init_global thy)))
+          |> List.filter (is_some o try (Syntax.check_term (Proof_Context.init_global thy)))
           |> take_random max_mutants
     val _ = map (fn t => Output.urgent_message ("MUTANT: " ^ Syntax.string_of_term_global thy t)) mutants
   in
@@ -490,7 +490,7 @@
 fun mutate_theorems_and_write_report thy mtds thms file_name =
   let
     val _ = Output.urgent_message "Starting Mutabelle..."
-    val ctxt = ProofContext.init_global thy
+    val ctxt = Proof_Context.init_global thy
     val path = Path.explode file_name
     (* for normal report: *)
     (*