src/HOL/Tools/Sledgehammer/sledgehammer_isar_proof.ML
changeset 66020 a31760eee09d
parent 61756 21c2b1f691d1
child 67399 eab6ce8368fa
--- a/src/HOL/Tools/Sledgehammer/sledgehammer_isar_proof.ML	Mon Jun 05 23:55:58 2017 +0200
+++ b/src/HOL/Tools/Sledgehammer/sledgehammer_isar_proof.ML	Tue Jun 06 13:13:25 2017 +0200
@@ -300,7 +300,7 @@
       (s ^ (term
             |> singleton (Syntax.uncheck_terms ctxt)
             |> annotate_types_in_term ctxt
-            |> with_vanilla_print_mode (Syntax.unparse_term ctxt #> Pretty.string_of)
+            |> Print_Mode.setmp [] (Syntax.unparse_term ctxt #> Pretty.string_of)
             |> simplify_spaces
             |> maybe_quote keywords),
        ctxt |> perhaps (try (Variable.auto_fixes term)))
@@ -320,7 +320,7 @@
 
     fun of_free (s, T) =
       maybe_quote keywords s ^ " :: " ^
-      maybe_quote keywords (simplify_spaces (with_vanilla_print_mode (Syntax.string_of_typ ctxt) T))
+      maybe_quote keywords (simplify_spaces (Print_Mode.setmp [] (Syntax.string_of_typ ctxt) T))
 
     fun add_frees xs (s, ctxt) =
       (s ^ space_implode " and " (map of_free xs), ctxt |> fold Variable.auto_fixes (map Free xs))