src/HOL/Nominal/nominal_inductive.ML
changeset 26939 1035c89b4c02
parent 26711 3a478bfa1650
child 27153 56b6cdce22f1
--- a/src/HOL/Nominal/nominal_inductive.ML	Sat May 17 23:53:20 2008 +0200
+++ b/src/HOL/Nominal/nominal_inductive.ML	Sun May 18 15:04:09 2008 +0200
@@ -614,7 +614,7 @@
       let
         fun eqvt_err s = error
           ("Could not prove equivariance for introduction rule\n" ^
-           Sign.string_of_term (theory_of_thm intr)
+           Syntax.string_of_term_global (theory_of_thm intr)
              (Logic.unvarify (prop_of intr)) ^ "\n" ^ s);
         val res = SUBPROOF (fn {prems, params, ...} =>
           let
@@ -630,7 +630,7 @@
       in
         case (Seq.pull res handle THM (s, _, _) => eqvt_err s) of
           NONE => eqvt_err ("Rule does not match goal\n" ^
-            Sign.string_of_term (theory_of_thm st) (hd (prems_of st)))
+            Syntax.string_of_term_global (theory_of_thm st) (hd (prems_of st)))
         | SOME (th, _) => Seq.single th
       end;
     val thss = map (fn atom =>