[1] goes after any attributes
authorblanchet
Thu, 26 Jul 2012 16:08:16 +0200
changeset 48535 619531d87ce4
parent 48534 2307efbfc554
child 48536 4e2ee88276d2
[1] goes after any attributes
src/HOL/Tools/try0.ML
--- a/src/HOL/Tools/try0.ML	Thu Jul 26 11:08:16 2012 +0200
+++ b/src/HOL/Tools/try0.ML	Thu Jul 26 16:08:16 2012 +0200
@@ -77,12 +77,13 @@
   if mode <> Auto_Try orelse run_if_auto_try then
     let val attrs = attrs_text attrs quad in
       do_generic timeout_opt
-                 (name ^ (if all_goals andalso
-                             nprems_of (#goal (Proof.goal st)) > 1 then
-                            "[1]"
-                          else
-                            "") ^
-                  attrs) I (#goal o Proof.goal)
+                 (name ^ attrs ^
+                  (if all_goals andalso
+                      nprems_of (#goal (Proof.goal st)) > 1 then
+                     " [1]"
+                   else
+                     ""))
+                 I (#goal o Proof.goal)
                  (apply_named_method_on_first_goal (name ^ attrs)
                                                    (Proof.theory_of st)) st
     end