prefer cat_lines;
authorwenzelm
Thu, 20 Feb 2014 19:38:34 +0100
changeset 55628 8103021024c1
parent 55627 95c8ef02f04b
child 55629 50f155005ea0
prefer cat_lines;
src/HOL/Tools/Nitpick/nitpick_mono.ML
src/HOL/Tools/Nitpick/nitpick_scope.ML
src/HOL/Tools/Predicate_Compile/predicate_compile.ML
src/Tools/coherent.ML
--- a/src/HOL/Tools/Nitpick/nitpick_mono.ML	Thu Feb 20 19:32:20 2014 +0100
+++ b/src/HOL/Tools/Nitpick/nitpick_mono.ML	Thu Feb 20 19:38:34 2014 +0100
@@ -531,7 +531,7 @@
        |> AList.group (op =)
        |> map (fn (a, xs) => string_for_annotation a ^ ": " ^
                              string_for_vars ", " (sort int_ord xs))
-       |> space_implode "\n"))
+       |> cat_lines))
 
 (* The ML solver timeout should correspond more or less to the overhead of invoking an external
    prover. *)
--- a/src/HOL/Tools/Nitpick/nitpick_scope.ML	Thu Feb 20 19:32:20 2014 +0100
+++ b/src/HOL/Tools/Nitpick/nitpick_scope.ML	Thu Feb 20 19:38:34 2014 +0100
@@ -209,7 +209,7 @@
          (if null iters then [] else ["iter: " ^ commas (map implode iters)]) @
          miscs of
       [] => "empty"
-    | lines => space_implode "\n" lines
+    | lines => cat_lines lines
   end
 
 fun scopes_equivalent (s1 : scope, s2 : scope) =
--- a/src/HOL/Tools/Predicate_Compile/predicate_compile.ML	Thu Feb 20 19:32:20 2014 +0100
+++ b/src/HOL/Tools/Predicate_Compile/predicate_compile.ML	Thu Feb 20 19:38:34 2014 +0100
@@ -25,7 +25,7 @@
 fun print_intross options thy msg intross =
   if show_intermediate_results options then
     tracing (msg ^
-      (space_implode "\n" (map
+      (cat_lines (map
         (fn (c, intros) => "Introduction rule(s) of " ^ c ^ ":\n" ^
            commas (map (Display.string_of_thm_global thy) intros)) intross)))
   else ()
@@ -34,8 +34,8 @@
   if show_intermediate_results options then
     map (fn (c, thms) =>
       "Constant " ^ c ^ " has specification:\n" ^
-        (space_implode "\n" (map (Display.string_of_thm_global thy) thms)) ^ "\n") specs
-    |> space_implode "\n" |> tracing
+        (cat_lines (map (Display.string_of_thm_global thy) thms)) ^ "\n") specs
+    |> cat_lines |> tracing
   else ()
 
 fun overload_const thy s = the_default s (Option.map fst (Axclass.inst_of_param thy s))
--- a/src/Tools/coherent.ML	Thu Feb 20 19:32:20 2014 +0100
+++ b/src/Tools/coherent.ML	Thu Feb 20 19:38:34 2014 +0100
@@ -119,7 +119,7 @@
 val show_facts = Unsynchronized.ref false;
 
 fun string_of_facts ctxt s facts =
-  space_implode "\n"
+  cat_lines
     (s :: map (Syntax.string_of_term ctxt)
       (map fst (sort (int_ord o pairself snd) (Net.content facts)))) ^ "\n\n";
 
@@ -175,8 +175,8 @@
 fun thm_of_cl_prf thy goal asms (ClPrf (th, (tye, env), insts, is, prfs)) =
   let
     val _ =
-      message (fn () => space_implode "\n"
-        ("asms:" :: map (Display.string_of_thm_global thy) asms) ^ "\n\n");
+      message (fn () =>
+        cat_lines ("asms:" :: map (Display.string_of_thm_global thy) asms) ^ "\n\n");
     val th' =
       Drule.implies_elim_list
         (Thm.instantiate