src/Pure/Isar/method.ML
changeset 15456 956d6acacf89
parent 14981 e73f8140af78
child 15531 08c8dad8e399
--- a/src/Pure/Isar/method.ML	Mon Jan 24 16:25:36 2005 +0100
+++ b/src/Pure/Isar/method.ML	Mon Jan 24 17:56:18 2005 +0100
@@ -487,8 +487,8 @@
 fun tactic txt ctxt = METHOD (fn facts =>
   (Context.use_mltext
     ("let fun tactic (ctxt: PureIsar.Proof.context) (facts: thm list) : tactic = \
-     \let val thm = PureIsar.ProofContext.get_thm_closure ctxt\n\
-     \  and thms = PureIsar.ProofContext.get_thms_closure ctxt in\n"
+     \let val thm = PureIsar.ProofContext.get_thm_closure ctxt o rpair None\n\
+     \  and thms = PureIsar.ProofContext.get_thms_closure ctxt o rpair None in\n"
      ^ txt ^
      "\nend in PureIsar.Method.set_tactic tactic end")
     false None;