src/Pure/Isar/method.ML
changeset 53044 be27b6be8027
parent 52732 b4da1f2ec73f
child 53168 d998de7f0efc
equal deleted inserted replaced
53043:8cbfbeb566a4 53044:be27b6be8027
    60   val this_text: text
    60   val this_text: text
    61   val done_text: text
    61   val done_text: text
    62   val sorry_text: bool -> text
    62   val sorry_text: bool -> text
    63   val finish_text: text option * bool -> text
    63   val finish_text: text option * bool -> text
    64   val print_methods: theory -> unit
    64   val print_methods: theory -> unit
       
    65   val check: theory -> xstring * Position.T -> string
    65   val intern: theory -> xstring -> string
    66   val intern: theory -> xstring -> string
    66   val defined: theory -> string -> bool
       
    67   val method: theory -> src -> Proof.context -> method
    67   val method: theory -> src -> Proof.context -> method
    68   val method_i: theory -> src -> Proof.context -> method
    68   val method_i: theory -> src -> Proof.context -> method
    69   val syntax: 'a context_parser -> src -> Proof.context -> 'a * Proof.context
    69   val syntax: 'a context_parser -> src -> Proof.context -> 'a * Proof.context
    70   val setup: binding -> (Proof.context -> method) context_parser -> string -> theory -> theory
    70   val setup: binding -> (Proof.context -> method) context_parser -> string -> theory -> theory
    71   val method_setup: bstring * Position.T -> Symbol_Pos.text * Position.T -> string ->
    71   val method_setup: bstring * Position.T -> Symbol_Pos.text * Position.T -> string ->
   329   |> Methods.map (Name_Space.define (Context.Theory thy) true (name, (meth, comment)) #> snd);
   329   |> Methods.map (Name_Space.define (Context.Theory thy) true (name, (meth, comment)) #> snd);
   330 
   330 
   331 
   331 
   332 (* get methods *)
   332 (* get methods *)
   333 
   333 
       
   334 fun check thy = #1 o Name_Space.check (Context.Theory thy) (Methods.get thy);
       
   335 
   334 val intern = Name_Space.intern o #1 o Methods.get;
   336 val intern = Name_Space.intern o #1 o Methods.get;
   335 val defined = Symtab.defined o #2 o Methods.get;
       
   336 
   337 
   337 fun method_i thy =
   338 fun method_i thy =
   338   let
   339   let
   339     val (space, tab) = Methods.get thy;
   340     val (space, tab) = Methods.get thy;
   340     fun meth src =
   341     fun meth src =