src/Pure/Isar/outer_syntax.ML
changeset 59083 88b0b1f28adc
parent 58999 ed09ae4ea2d8
child 59923 b21c82422d65
equal deleted inserted replaced
59082:25501ba956ac 59083:88b0b1f28adc
    17     (local_theory -> local_theory) parser -> unit
    17     (local_theory -> local_theory) parser -> unit
    18   val local_theory_to_proof': command_spec -> string ->
    18   val local_theory_to_proof': command_spec -> string ->
    19     (bool -> local_theory -> Proof.state) parser -> unit
    19     (bool -> local_theory -> Proof.state) parser -> unit
    20   val local_theory_to_proof: command_spec -> string ->
    20   val local_theory_to_proof: command_spec -> string ->
    21     (local_theory -> Proof.state) parser -> unit
    21     (local_theory -> Proof.state) parser -> unit
    22   val scan: Keyword.keywords -> Position.T -> string -> Token.T list
       
    23   val parse: theory -> Position.T -> string -> Toplevel.transition list
    22   val parse: theory -> Position.T -> string -> Toplevel.transition list
    24   val parse_tokens: theory -> Token.T list -> Toplevel.transition list
    23   val parse_tokens: theory -> Token.T list -> Toplevel.transition list
    25   val parse_spans: Token.T list -> Command_Span.span list
    24   val parse_spans: Token.T list -> Command_Span.span list
    26   val side_comments: Token.T list -> Token.T list
    25   val side_comments: Token.T list -> Token.T list
    27   val command_reports: theory -> Token.T -> Position.report_text list
    26   val command_reports: theory -> Token.T -> Position.report_text list
   145 val local_theory_to_proof = local_theory_command Toplevel.local_theory_to_proof;
   144 val local_theory_to_proof = local_theory_command Toplevel.local_theory_to_proof;
   146 
   145 
   147 
   146 
   148 
   147 
   149 (** toplevel parsing **)
   148 (** toplevel parsing **)
   150 
       
   151 (* scan tokens *)
       
   152 
       
   153 fun scan keywords pos =
       
   154   Source.of_string #>
       
   155   Symbol.source #>
       
   156   Token.source keywords pos #>
       
   157   Source.exhaust;
       
   158 
       
   159 
   149 
   160 (* parse commands *)
   150 (* parse commands *)
   161 
   151 
   162 local
   152 local
   163 
   153