src/HOL/TPTP/MaSh_Export.thy
changeset 50966 b85cb3049df9
parent 50964 2a990baa09af
child 51027 0f817f80bcca
equal deleted inserted replaced
50965:7a7d1418301e 50966:b85cb3049df9
   103       (prefix ^ "mash_prover_commands")
   103       (prefix ^ "mash_prover_commands")
   104 else
   104 else
   105   ()
   105   ()
   106 *}
   106 *}
   107 
   107 
       
   108 ML {*
       
   109 if do_it then
       
   110   generate_mesh_suggestions max_suggestions (prefix ^ "mash_prover_suggestions")
       
   111       (prefix ^ "mepo_suggestions") (prefix ^ "mesh_prover_suggestions")
       
   112 else
       
   113   ()
       
   114 *}
       
   115 
   108 end
   116 end