method_setup: thms closure;
authorwenzelm
Sat, 02 Sep 2000 21:53:03 +0200
changeset 9810 7e785df2b76a
parent 9809 58e9d55a9f88
child 9811 39ffdb8cab03
method_setup: thms closure;
src/Pure/Isar/isar_thy.ML
--- a/src/Pure/Isar/isar_thy.ML	Sat Sep 02 21:52:33 2000 +0200
+++ b/src/Pure/Isar/isar_thy.ML	Sat Sep 02 21:53:03 2000 +0200
@@ -558,7 +558,9 @@
 
 fun method_setup ((name, txt, cmt), comment_ignore) =
   Context.use_let
-    "val method: bstring * (Args.src -> Proof.context -> Proof.method) * string"
+    "val thm = PureThy.get_thm_closure (Context.the_context ());\n\
+    \val thms = PureThy.get_thms_closure (Context.the_context ());\n\
+    \val method: bstring * (Args.src -> Proof.context -> Proof.method) * string"
     "PureIsar.Method.add_method method"
     ("(" ^ quote name ^ ", " ^ txt ^ ", " ^ quote cmt ^ ")");