src/Pure/Tools/rail.ML
changeset 67381 146757999c8d
parent 67147 dea94b1aabc3
child 67386 998e01d6f8fd
--- a/src/Pure/Tools/rail.ML	Mon Jan 08 22:36:02 2018 +0100
+++ b/src/Pure/Tools/rail.ML	Mon Jan 08 23:45:43 2018 +0100
@@ -17,7 +17,7 @@
     Terminal of bool * string |
     Antiquote of bool * Antiquote.antiq
   val read: Proof.context -> Input.source -> (string Antiquote.antiquote * rail) list
-  val output_rules: Toplevel.state -> (string Antiquote.antiquote * rail) list -> string
+  val output_rules: Proof.context -> (string Antiquote.antiquote * rail) list -> string
 end;
 
 structure Rail: RAIL =
@@ -330,9 +330,9 @@
 
 in
 
-fun output_rules state rules =
+fun output_rules ctxt rules =
   let
-    val output_antiq = Thy_Output.eval_antiquote state o Antiquote.Antiq;
+    val output_antiq = Thy_Output.eval_antiquote ctxt o Antiquote.Antiq;
     fun output_text b s =
       Output.output s
       |> b ? enclose "\\isakeyword{" "}"
@@ -375,7 +375,7 @@
 
 val _ = Theory.setup
   (Thy_Output.antiquotation \<^binding>\<open>rail\<close> (Scan.lift Args.text_input)
-    (fn {state, context, ...} => output_rules state o read context));
+    (fn {context = ctxt, ...} => output_rules ctxt o read ctxt));
 
 end;