src/Pure/Isar/token.ML
changeset 58865 ce8d13995516
parent 58864 505a8150368a
child 58903 38c72f5f6c2e
--- a/src/Pure/Isar/token.ML	Sat Nov 01 19:33:51 2014 +0100
+++ b/src/Pure/Isar/token.ML	Sat Nov 01 19:47:48 2014 +0100
@@ -87,7 +87,7 @@
       (Symbol_Pos.T, Position.T * (Symbol.symbol, 'a) Source.source) Source.source) Source.source
   type 'a parser = T list -> 'a * T list
   type 'a context_parser = Context.generic * T list -> 'a * (Context.generic * T list)
-  val read: Scan.lexicon -> 'a parser -> Symbol_Pos.T list * Position.T -> 'a list
+  val read: Scan.lexicon -> 'a parser -> Symbol_Pos.T list -> 'a list
   val read_antiq: Scan.lexicon -> 'a parser -> Symbol_Pos.T list * Position.T -> 'a
   val syntax_generic: 'a context_parser -> src -> Context.generic -> 'a * Context.generic
   val syntax: 'a context_parser -> src -> Proof.context -> 'a * Proof.context
@@ -582,7 +582,7 @@
 
 (* read source *)
 
-fun read lex scan (syms, pos) =
+fun read lex scan syms =
   Source.of_list syms
   |> source' true (K (lex, Scan.empty_lexicon))
   |> source_proper
@@ -594,7 +594,7 @@
     fun err msg =
       cat_error msg ("Malformed antiquotation" ^ Position.here pos ^ ":\n" ^
         "@{" ^ Symbol_Pos.content syms ^ "}");
-    val res = read lex scan (syms, pos) handle ERROR msg => err msg;
+    val res = read lex scan syms handle ERROR msg => err msg;
   in (case res of [x] => x | _ => err "") end;