src/HOL/Tools/Sledgehammer/sledgehammer_proof_methods.ML
changeset 55451 ea1d9408a233
parent 55323 253a029335a2
child 55452 29ec8680e61f
equal deleted inserted replaced
55450:9eddc17749f7 55451:ea1d9408a233
   181       | Not_Played => (false, NONE))
   181       | Not_Played => (false, NONE))
   182 
   182 
   183     val try_line =
   183     val try_line =
   184       map fst extra
   184       map fst extra
   185       |> proof_method_command meth subgoal subgoal_count (map fst chained) num_chained
   185       |> proof_method_command meth subgoal subgoal_count (map fst chained) num_chained
   186       |> (if failed then
   186       |> (if failed then enclose "One-line proof reconstruction failed: " "."
   187             enclose "One-line proof reconstruction failed: "
   187           else try_command_line banner ext_time)
   188               ".\n(Invoking \"sledgehammer\" with \"[strict]\" might solve this.)"
       
   189           else
       
   190             try_command_line banner ext_time)
       
   191   in
   188   in
   192     try_line ^ minimize_line minimize_command (map fst (extra @ chained))
   189     try_line ^ minimize_line minimize_command (map fst (extra @ chained))
   193   end
   190   end
   194 
   191 
   195 (* Makes proof methods as silent as possible. The "set_visible" calls suppresses "Unification bound
   192 (* Makes proof methods as silent as possible. The "set_visible" calls suppresses "Unification bound