Fri, 03 Oct 2008 20:10:43 +0200 wenzelm updated to new AtpManager;
Fri, 03 Oct 2008 19:35:18 +0200 wenzelm operate on Proof.state, not Toplevel.state;
Fri, 03 Oct 2008 19:35:17 +0200 wenzelm misc simplifcation and tuning;
Fri, 03 Oct 2008 19:35:16 +0200 wenzelm perform atp_setups here;
Fri, 03 Oct 2008 19:35:15 +0200 wenzelm updated generated file;
Fri, 03 Oct 2008 19:35:14 +0200 wenzelm removed HOL-Plain -- already included in HOL;
Fri, 03 Oct 2008 19:17:37 +0200 wenzelm removed spurious ResAtp.set_prover;
Fri, 03 Oct 2008 17:07:41 +0200 wenzelm simplified thread creation via SimpleThread;
Fri, 03 Oct 2008 17:07:39 +0200 wenzelm simplified thread creation via SimpleThread;
Fri, 03 Oct 2008 16:37:09 +0200 wenzelm version of sledgehammer using threads instead of processes, misc cleanup;
Fri, 03 Oct 2008 15:20:33 +0200 wenzelm removed old/unused setup of raw ATP oracles;
Fri, 03 Oct 2008 14:07:41 +0200 wenzelm tuned;
Fri, 03 Oct 2008 14:06:19 +0200 wenzelm Vampire wrapper script for remote SystemOnTPTP service (by Fabian Immler);
Fri, 03 Oct 2008 13:21:01 +0200 wenzelm added PROOFGENERAL_EMACS, with attempt to find Carbon Emacs;
Fri, 03 Oct 2008 00:21:48 +0200 wenzelm tuned tracing;
Fri, 03 Oct 2008 00:12:13 +0200 wenzelm slower heartbeat;
Thu, 02 Oct 2008 23:52:12 +0200 wenzelm added simple heartbeat thread;
Thu, 02 Oct 2008 23:52:10 +0200 wenzelm time factor: one more digit;
Thu, 02 Oct 2008 23:30:44 +0200 wenzelm more tuning of tracing messages;
Thu, 02 Oct 2008 22:09:22 +0200 wenzelm include factor in timing report;
Thu, 02 Oct 2008 21:21:21 +0200 wenzelm with_attributes: enforces InterruptAsynch => InterruptAsynchOnce to avoid race condition;
Thu, 02 Oct 2008 19:59:01 +0200 wenzelm tracing: ignore failure of any kind;
Thu, 02 Oct 2008 19:59:00 +0200 wenzelm tuned SYNCHRONIZED: outermost Exn.release;
Thu, 02 Oct 2008 19:38:48 +0200 wenzelm program wrapper: controlled_execution ensures proper thread attributes (global default is unsafe due to InterruptAsynch;
Thu, 02 Oct 2008 17:18:36 +0200 haftmann added partiality section
Thu, 02 Oct 2008 17:18:22 +0200 haftmann corrected class antiquotation
Thu, 02 Oct 2008 14:22:45 +0200 wenzelm max_threads_value always 1 for dummy version;
Thu, 02 Oct 2008 14:22:44 +0200 wenzelm simplified Exn.EXCEPTIONS, flatten nested occurrences;
Thu, 02 Oct 2008 14:22:40 +0200 wenzelm simplified Exn.EXCEPTIONS;
Thu, 02 Oct 2008 14:22:36 +0200 wenzelm major cleanup of hoare_tac.ML: just one copy for Hoare.thy and HoareAbort.thy (only 1 line different), refrain from inspecting the main goal, proper context;
Thu, 02 Oct 2008 13:07:33 +0200 haftmann tuned
Thu, 02 Oct 2008 12:17:20 +0200 berghofe Yet another proof of Newman's lemma, this time using the coherent logic prover.
Wed, 01 Oct 2008 22:33:29 +0200 wenzelm unit_source: more rigid parsing, stop after final qed;
Wed, 01 Oct 2008 22:33:28 +0200 wenzelm excursion/unit_result: no print for forked end, finish into global theory, pick resul from presentation context;
Wed, 01 Oct 2008 22:33:24 +0200 wenzelm replaced can_defer by is_relevant (negation);
Wed, 01 Oct 2008 20:02:37 +0200 wenzelm datatype transition: internal trans field is maintained in reverse order;
Wed, 01 Oct 2008 18:16:14 +0200 wenzelm future_proof: protect conclusion of deferred proof state;
Wed, 01 Oct 2008 18:16:10 +0200 wenzelm future_schedule: back to one group for all loader tasks;
Wed, 01 Oct 2008 14:17:06 +0200 wenzelm tuned comments;
Wed, 01 Oct 2008 13:33:54 +0200 haftmann fixed
Wed, 01 Oct 2008 12:18:18 +0200 wenzelm renamed promise to future, tuned related interfaces;
Wed, 01 Oct 2008 12:00:05 +0200 wenzelm more robust treatment of Interrupt (cf. exn.ML);
Wed, 01 Oct 2008 12:00:04 +0200 wenzelm more robust treatment of Interrupt;
Wed, 01 Oct 2008 12:00:02 +0200 wenzelm more robust treatment of Interrupt (cf. exn.ML);
Wed, 01 Oct 2008 12:00:01 +0200 wenzelm removed release_results (cf. Exn.release_all, Exn.release_first);
Wed, 01 Oct 2008 12:00:00 +0200 wenzelm more precise join_futures, improved termination;
Wed, 01 Oct 2008 08:42:42 +0200 haftmann added more_antiquote.ML
Wed, 01 Oct 2008 00:09:51 +0200 kleing extract Isabelle dist name correctly
Tue, 30 Sep 2008 23:31:40 +0200 wenzelm unit_source: explicit treatment of 'oops' proofs;
Tue, 30 Sep 2008 23:31:38 +0200 wenzelm promise_proof: proper statement with empty vars;
Tue, 30 Sep 2008 23:31:36 +0200 wenzelm load_thy: more precise treatment of improper cmd or proof (notably 'oops');
Tue, 30 Sep 2008 22:02:55 +0200 wenzelm schedule_tasks: single theory is loaded concurrently as well (cf. concurrent Toplevel.excursion);
Tue, 30 Sep 2008 22:02:53 +0200 wenzelm added unit_source: commands with proof;
Tue, 30 Sep 2008 22:02:51 +0200 wenzelm begin_proof: avoid race condition wrt. skip_proofs flag;
Tue, 30 Sep 2008 22:02:50 +0200 wenzelm load_thy: Toplevel.excursion based on units of command/proof pairs;
Tue, 30 Sep 2008 22:02:47 +0200 wenzelm more command categories;
Tue, 30 Sep 2008 22:02:45 +0200 wenzelm renamed Future.fork_irrelevant to Future.fork_background;
Tue, 30 Sep 2008 22:02:44 +0200 wenzelm export explicit joint_futures, removed Theory.at_end hook;
Tue, 30 Sep 2008 14:30:44 +0200 haftmann tuned
Tue, 30 Sep 2008 14:19:28 +0200 wenzelm turned process_thy into present_thy, which merely does presentation (wrt. persistent intermediate states);
(0) -10000 -3000 -1000 -300 -100 -60 +60 +100 +300 +1000 +3000 +10000 +30000 tip