src/Pure/sign.ML
changeset 42247 12fe41a92cd5
parent 42224 578a51fae383
child 42268 01401287c3f7
--- a/src/Pure/sign.ML	Wed Apr 06 13:27:59 2011 +0200
+++ b/src/Pure/sign.ML	Wed Apr 06 13:33:46 2011 +0200
@@ -95,15 +95,14 @@
     (string * (term list -> term)) list *
     (string * (term list -> term)) list *
     (string * (Ast.ast list -> Ast.ast)) list -> theory -> theory
-  val add_trfunsT:
-    (string * (bool -> typ -> term list -> term)) list -> theory -> theory
+  val add_trfunsT: (string * (typ -> term list -> term)) list -> theory -> theory
   val add_advanced_trfuns:
     (string * (Proof.context -> Ast.ast list -> Ast.ast)) list *
     (string * (Proof.context -> term list -> term)) list *
     (string * (Proof.context -> term list -> term)) list *
     (string * (Proof.context -> Ast.ast list -> Ast.ast)) list -> theory -> theory
   val add_advanced_trfunsT:
-    (string * (Proof.context -> bool -> typ -> term list -> term)) list -> theory -> theory
+    (string * (Proof.context -> typ -> term list -> term)) list -> theory -> theory
   val add_tokentrfuns:
     (string * string * (Proof.context -> string -> Pretty.T)) list -> theory -> theory
   val add_mode_tokentrfuns: string -> (string * (Proof.context -> string -> Pretty.T)) list