src/Pure/Isar/toplevel.ML
changeset 12881 eeb36b66480e
parent 12423 7fd447422dee
child 12987 b6db96775e52
equal deleted inserted replaced
12880:21485940c8b9 12881:eeb36b66480e
   383   | exn_message (ProofContext.CONTEXT (msg, _)) = msg
   383   | exn_message (ProofContext.CONTEXT (msg, _)) = msg
   384   | exn_message (Proof.STATE (msg, _)) = msg
   384   | exn_message (Proof.STATE (msg, _)) = msg
   385   | exn_message (ProofHistory.FAIL msg) = msg
   385   | exn_message (ProofHistory.FAIL msg) = msg
   386   | exn_message (Attrib.ATTRIB_FAIL info) = fail_message "attribute" info
   386   | exn_message (Attrib.ATTRIB_FAIL info) = fail_message "attribute" info
   387   | exn_message (Method.METHOD_FAIL info) = fail_message "method" info
   387   | exn_message (Method.METHOD_FAIL info) = fail_message "method" info
   388   | exn_message (Comment.OUTPUT_FAIL info) = fail_message "antiquotation" info
   388   | exn_message (Antiquote.ANTIQUOTE_FAIL info) = fail_message "antiquotation" info
   389   | exn_message (Syntax.AST (msg, _)) = raised_msg "AST" msg
   389   | exn_message (Syntax.AST (msg, _)) = raised_msg "AST" msg
   390   | exn_message (TYPE (msg, _, _)) = raised_msg "TYPE" msg
   390   | exn_message (TYPE (msg, _, _)) = raised_msg "TYPE" msg
   391   | exn_message (TERM (msg, _)) = raised_msg "TERM" msg
   391   | exn_message (TERM (msg, _)) = raised_msg "TERM" msg
   392   | exn_message (THM (msg, _, _)) = raised_msg "THM" msg
   392   | exn_message (THM (msg, _, _)) = raised_msg "THM" msg
   393   | exn_message Library.OPTION = raised "Library.OPTION"
   393   | exn_message Library.OPTION = raised "Library.OPTION"
   469 
   469 
   470 (* the Isar source of transitions *)
   470 (* the Isar source of transitions *)
   471 
   471 
   472 type isar =
   472 type isar =
   473   (transition, (transition option,
   473   (transition, (transition option,
   474     (OuterLex.token, (OuterLex.token,
   474     (OuterLex.token, (OuterLex.token option, (OuterLex.token, (OuterLex.token,
   475       Position.T * (Symbol.symbol, (string, unit) Source.source) Source.source)
   475       Position.T * (Symbol.symbol, (string, unit) Source.source) Source.source)
   476           Source.source) Source.source) Source.source) Source.source;
   476           Source.source) Source.source) Source.source) Source.source) Source.source) Source.source;
   477 
   477 
   478 
   478 
   479 (* apply transformers to global state *)
   479 (* apply transformers to global state *)
   480 
   480 
   481 nonfix >>;
   481 nonfix >>;