src/HOL/Tools/TFL/tfl.ML
changeset 26928 ca87aff1ad2d
parent 26177 6b127c056e83
child 26939 1035c89b4c02
--- a/src/HOL/Tools/TFL/tfl.ML	Fri May 16 23:25:37 2008 +0200
+++ b/src/HOL/Tools/TFL/tfl.ML	Sat May 17 13:54:30 2008 +0200
@@ -298,7 +298,7 @@
             raise TFL_ERR "no_repeat_vars"
                           (quote (#1 (dest_Free v)) ^
                           " occurs repeatedly in the pattern " ^
-                          quote (string_of_cterm (Thry.typecheck thy pat)))
+                          quote (Display.string_of_cterm (Thry.typecheck thy pat)))
          else check rst
  in check (FV_multiset pat)
  end;
@@ -532,7 +532,7 @@
      val (extractants,TCl) = ListPair.unzip extracta
      val dummy = if !trace
                  then (writeln "Extractants = ";
-                       prths extractants;
+                       Display.prths extractants;
                        ())
                  else ()
      val TCs = foldr (gen_union (op aconv)) [] TCl
@@ -553,7 +553,7 @@
        |> PureThy.add_defs_i false
             [Thm.no_attributes (fid ^ "_def", defn)]
      val def = Thm.freezeT def0;
-     val dummy = if !trace then writeln ("DEF = " ^ string_of_thm def)
+     val dummy = if !trace then writeln ("DEF = " ^ Display.string_of_thm def)
                            else ()
      (* val fconst = #lhs(S.dest_eq(concl def))  *)
      val tych = Thry.typecheck theory
@@ -562,7 +562,7 @@
      val baz = R.DISCH_ALL
                  (fold_rev R.DISCH full_rqt_prop
                   (R.LIST_CONJ extractants))
-     val dum = if !trace then writeln ("baz = " ^ string_of_thm baz)
+     val dum = if !trace then writeln ("baz = " ^ Display.string_of_thm baz)
                            else ()
      val f_free = Free (fid, fastype_of f)  (*'cos f is a Const*)
      val SV' = map tych SV;
@@ -911,11 +911,11 @@
 
 
 fun trace_thms s L =
-  if !trace then writeln (cat_lines (s :: map string_of_thm L))
+  if !trace then writeln (cat_lines (s :: map Display.string_of_thm L))
   else ();
 
 fun trace_cterms s L =
-  if !trace then writeln (cat_lines (s :: map string_of_cterm L))
+  if !trace then writeln (cat_lines (s :: map Display.string_of_cterm L))
   else ();;