token translations: context dependent, result Pretty.T;
authorwenzelm
Thu, 17 Apr 2008 16:30:47 +0200
changeset 26701 341c4d51d1c2
parent 26700 493db7848904
child 26702 a079f8f0080b
token translations: context dependent, result Pretty.T;
src/Pure/sign.ML
--- a/src/Pure/sign.ML	Thu Apr 17 16:30:45 2008 +0200
+++ b/src/Pure/sign.ML	Thu Apr 17 16:30:47 2008 +0200
@@ -135,8 +135,8 @@
   val add_advanced_trfunsT:
     (string * (Proof.context -> bool -> typ -> term list -> term)) list -> theory -> theory
   val add_tokentrfuns:
-    (string * string * (string -> output * int)) list -> theory -> theory
-  val add_mode_tokentrfuns: string -> (string * (string -> output * int)) list
+    (string * string * (Proof.context -> string -> Pretty.T)) list -> theory -> theory
+  val add_mode_tokentrfuns: string -> (string * (Proof.context -> string -> Pretty.T)) list
     -> theory -> theory
   val add_trrules: (xstring * string) Syntax.trrule list -> theory -> theory
   val del_trrules: (xstring * string) Syntax.trrule list -> theory -> theory