src/Pure/Isar/method.ML
changeset 25699 891fe6b71d3b
parent 25270 2ed7b34f58e6
child 25957 2cfb703fa8d8
--- 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));