wenzelm [Fri, 03 Oct 2008 20:10:43 +0200] rev 28486
updated to new AtpManager;
wenzelm [Fri, 03 Oct 2008 19:35:18 +0200] rev 28485
operate on Proof.state, not Toplevel.state;
moved setup to ATP_Linkup.thy;
wenzelm [Fri, 03 Oct 2008 19:35:17 +0200] rev 28484
misc simplifcation and tuning;
no export of structure Provers;
added add_provers, print_provers;
operate on Proof.state, not Toplevel.state;
use Time.+ etc. to make SML/XL of NJ happy;
explicit Isar commands 'atp_kill', 'atp_info', 'print_atps';
wenzelm [Fri, 03 Oct 2008 19:35:16 +0200] rev 28483
perform atp_setups here;
wenzelm [Fri, 03 Oct 2008 19:35:15 +0200] rev 28482
updated generated file;
wenzelm [Fri, 03 Oct 2008 19:35:14 +0200] rev 28481
removed HOL-Plain -- already included in HOL;
wenzelm [Fri, 03 Oct 2008 19:17:37 +0200] rev 28480
removed spurious ResAtp.set_prover;
wenzelm [Fri, 03 Oct 2008 17:07:41 +0200] rev 28479
simplified thread creation via SimpleThread;
wenzelm [Fri, 03 Oct 2008 17:07:39 +0200] rev 28478
simplified thread creation via SimpleThread;
managing_thread: option type (fork of inactive thread assumes threads are available in the first place);
wenzelm [Fri, 03 Oct 2008 16:37:09 +0200] rev 28477
version of sledgehammer using threads instead of processes, misc cleanup;
(by Fabian Immler);