src/ZF/Datatype_ZF.thy
changeset 26928 ca87aff1ad2d
parent 26480 544cef16045b
child 26939 1035c89b4c02
--- a/src/ZF/Datatype_ZF.thy	Fri May 16 23:25:37 2008 +0200
+++ b/src/ZF/Datatype_ZF.thy	Sat May 17 13:54:30 2008 +0200
@@ -72,7 +72,7 @@
 
  fun proc sg ss old =
    let val _ = if !trace then writeln ("data_free: OLD = " ^ 
-                                       string_of_cterm (cterm_of sg old))
+                                       Display.string_of_cterm (cterm_of sg old))
                else ()
        val (lhs,rhs) = FOLogic.dest_eq old
        val (lhead, largs) = strip_comb lhs
@@ -90,7 +90,7 @@
                else Const("False",FOLogic.oT)
            else raise Match
        val _ = if !trace then 
-                 writeln ("NEW = " ^ string_of_cterm (Thm.cterm_of sg new))
+                 writeln ("NEW = " ^ Display.string_of_cterm (Thm.cterm_of sg new))
                else ();
        val goal = Logic.mk_equals (old, new)
        val thm = Goal.prove (Simplifier.the_context ss) [] [] goal