src/Pure/Isar/method.ML
changeset 61917 35ec3757d3c1
parent 61843 1803599838a6
child 62795 063d2f23cdf6
equal deleted inserted replaced
61915:e9812a95d108 61917:35ec3757d3c1
    71   val finish_text: text option * bool -> text
    71   val finish_text: text option * bool -> text
    72   val print_methods: bool -> Proof.context -> unit
    72   val print_methods: bool -> Proof.context -> unit
    73   val check_name: Proof.context -> xstring * Position.T -> string
    73   val check_name: Proof.context -> xstring * Position.T -> string
    74   val check_src: Proof.context -> Token.src -> Token.src
    74   val check_src: Proof.context -> Token.src -> Token.src
    75   val check_text: Proof.context -> text -> text
    75   val check_text: Proof.context -> text -> text
       
    76   val checked_text: text -> bool
    76   val method_syntax: (Proof.context -> method) context_parser ->
    77   val method_syntax: (Proof.context -> method) context_parser ->
    77     Token.src -> Proof.context -> method
    78     Token.src -> Proof.context -> method
    78   val setup: binding -> (Proof.context -> method) context_parser -> string -> theory -> theory
    79   val setup: binding -> (Proof.context -> method) context_parser -> string -> theory -> theory
    79   val local_setup: binding -> (Proof.context -> method) context_parser -> string ->
    80   val local_setup: binding -> (Proof.context -> method) context_parser -> string ->
    80     local_theory -> local_theory
    81     local_theory -> local_theory
   436   #1 o Token.check_src ctxt (get_methods o Context.Proof);
   437   #1 o Token.check_src ctxt (get_methods o Context.Proof);
   437 
   438 
   438 fun check_text ctxt (Source src) = Source (check_src ctxt src)
   439 fun check_text ctxt (Source src) = Source (check_src ctxt src)
   439   | check_text _ (Basic m) = Basic m
   440   | check_text _ (Basic m) = Basic m
   440   | check_text ctxt (Combinator (x, y, body)) = Combinator (x, y, map (check_text ctxt) body);
   441   | check_text ctxt (Combinator (x, y, body)) = Combinator (x, y, map (check_text ctxt) body);
       
   442 
       
   443 fun checked_text (Source src) = Token.checked_src src
       
   444   | checked_text (Basic _) = true
       
   445   | checked_text (Combinator (_, _, body)) = forall checked_text body;
   441 
   446 
   442 
   447 
   443 (* method setup *)
   448 (* method setup *)
   444 
   449 
   445 fun method_syntax scan src ctxt : method =
   450 fun method_syntax scan src ctxt : method =