named some critical sections;
authorwenzelm
Tue, 18 Dec 2007 19:54:33 +0100
changeset 25699 891fe6b71d3b
parent 25698 8c335b4641a5
child 25700 185ea28035ac
named some critical sections;
src/Pure/Isar/method.ML
src/Pure/Thy/thm_database.ML
--- a/src/Pure/Isar/method.ML	Tue Dec 18 19:54:32 2007 +0100
+++ b/src/Pure/Isar/method.ML	Tue Dec 18 19:54:33 2007 +0100
@@ -351,7 +351,7 @@
 val tactic_ref = ref ((fn _ => raise Match): Proof.context -> thm list -> tactic);
 fun set_tactic f = tactic_ref := f;
 
-fun ml_tactic txt ctxt = CRITICAL (fn () =>
+fun ml_tactic txt ctxt = NAMED_CRITICAL "ML" (fn () =>
   (ML_Context.use_mltext
     ("let fun tactic (ctxt: Proof.context) (facts: thm list) : tactic =\n"
       ^ txt ^ "\nin Method.set_tactic tactic end") false (SOME (Context.Proof ctxt));
--- a/src/Pure/Thy/thm_database.ML	Tue Dec 18 19:54:32 2007 +0100
+++ b/src/Pure/Thy/thm_database.ML	Tue Dec 18 19:54:33 2007 +0100
@@ -51,14 +51,14 @@
 fun ml_store_thm (name, thm) =
   let val thm' = store_thm (name, thm) in
     if warn_ml name then ()
-    else CRITICAL (fn () => (qed_thms := [thm'];
+    else NAMED_CRITICAL "ML" (fn () => (qed_thms := [thm'];
       use_text_verbose ("val " ^ name ^ " = hd (! ThmDatabase.qed_thms);")))
   end;
 
 fun ml_store_thms (name, thms) =
   let val thms' = store_thms (name, thms) in
     if warn_ml name then ()
-    else CRITICAL (fn () => (qed_thms := thms';
+    else NAMED_CRITICAL "ML" (fn () => (qed_thms := thms';
       use_text_verbose ("val " ^ name ^ " = ! ThmDatabase.qed_thms;")))
   end;