added intern, defined;
authorwenzelm
Wed, 14 May 2008 20:30:29 +0200
changeset 26892 9454a8bd1114
parent 26891 bfa1944e5238
child 26893 44d9960d3587
added intern, defined;
src/Pure/Isar/method.ML
--- a/src/Pure/Isar/method.ML	Wed May 14 20:30:05 2008 +0200
+++ b/src/Pure/Isar/method.ML	Wed May 14 20:30:29 2008 +0200
@@ -70,6 +70,8 @@
   val done_text: text
   val sorry_text: bool -> text
   val finish_text: text option * bool -> Position.T -> text
+  val intern: theory -> xstring -> string
+  val defined: theory -> string -> bool
   val method: theory -> src -> Proof.context -> method
   val method_i: theory -> src -> Proof.context -> method
   val add_methods: (bstring * (src -> Proof.context -> method) * string) list
@@ -424,6 +426,9 @@
 
 (* get methods *)
 
+val intern = NameSpace.intern o #1 o Methods.get;
+val defined = Symtab.defined o #2 o Methods.get;
+
 fun method_i thy =
   let
     val meths = #2 (Methods.get thy);