src/Pure/Isar/method.ML
changeset 26892 9454a8bd1114
parent 26762 78ed28528ca6
child 27235 134991516430
--- 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);