nipkow [Tue, 05 Mar 2013 10:16:15 +0100] rev 51334
more lemmas about intervals
wenzelm [Mon, 04 Mar 2013 17:32:10 +0100] rev 51333
merged
wenzelm [Mon, 04 Mar 2013 15:03:46 +0100] rev 51332
refined parallel_proofs = 2: fork whole Isar sub-proofs, not just terminal ones;
refined parallel_proofs = 3: fork terminal proofs, as poor man's parallelization in interactive mode;
wenzelm [Mon, 04 Mar 2013 11:36:16 +0100] rev 51331
join all proofs before scheduling present phase (ordered according to weight);
tuned;
wenzelm [Mon, 04 Mar 2013 10:02:58 +0100] rev 51330
more explicit datatype result;
hoelzl [Wed, 20 Feb 2013 12:04:42 +0100] rev 51329
split dense into inner_dense_order and no_top/no_bot
hoelzl [Wed, 20 Feb 2013 12:04:42 +0100] rev 51328
move auxiliary lemmas from Library/Extended_Reals to HOL image
traytel [Mon, 04 Mar 2013 09:57:54 +0100] rev 51327
tuned (extend datatype to inline option)
wenzelm [Sun, 03 Mar 2013 18:50:46 +0100] rev 51326
prefer more systematic Future.flat;
wenzelm [Sun, 03 Mar 2013 17:34:42 +0100] rev 51325
more uniform Future.map: always internalize failure;
added Future.flat as fast-path operation;
wenzelm [Sun, 03 Mar 2013 14:29:30 +0100] rev 51324
uniform treatment of global/local proofs;
tuned;
wenzelm [Sun, 03 Mar 2013 13:57:03 +0100] rev 51323
tuned;
wenzelm [Sun, 03 Mar 2013 13:43:57 +0100] rev 51322
clarified Toplevel.element_result wrt. Toplevel.is_ignored;
wenzelm [Sun, 03 Mar 2013 13:23:06 +0100] rev 51321
more Thy_Syntax.element operations;
traytel [Fri, 01 Mar 2013 22:15:31 +0100] rev 51320
coercion-invariant arguments at work
traytel [Fri, 01 Mar 2013 22:15:31 +0100] rev 51319
constants with coercion-invariant arguments (possibility to disable/reenable
coercions under certain constants, necessary for the forthcoming logically
unspecified control structures for case translations)
wenzelm [Thu, 28 Feb 2013 21:11:07 +0100] rev 51318
simplified Proof.future_proof;
wenzelm [Thu, 28 Feb 2013 18:35:31 +0100] rev 51317
provide explicit dummy names (cf. dfe469293eb4);
wenzelm [Thu, 28 Feb 2013 17:38:35 +0100] rev 51316
discontinued empty name bindings in 'axiomatization';
wenzelm [Thu, 28 Feb 2013 17:14:55 +0100] rev 51315
provide common HOLogic.conj_conv and HOLogic.eq_conv;
wenzelm [Thu, 28 Feb 2013 16:54:52 +0100] rev 51314
just one HOLogic.Trueprop_conv, with regular exception CTERM;
tuned;
wenzelm [Thu, 28 Feb 2013 16:38:17 +0100] rev 51313
discontinued obsolete 'axioms' command;
wenzelm [Thu, 28 Feb 2013 16:19:08 +0100] rev 51312
more robust build error handling, e.g. missing outer syntax commands;
wenzelm [Thu, 28 Feb 2013 14:29:54 +0100] rev 51311
eliminated legacy 'axioms';
wenzelm [Thu, 28 Feb 2013 14:24:21 +0100] rev 51310
eliminated legacy 'axioms';
wenzelm [Thu, 28 Feb 2013 14:22:14 +0100] rev 51309
eliminated legacy 'axioms';
wenzelm [Thu, 28 Feb 2013 14:10:54 +0100] rev 51308
eliminated legacy 'axioms';
wenzelm [Thu, 28 Feb 2013 13:54:45 +0100] rev 51307
eliminated legacy 'axioms';
wenzelm [Thu, 28 Feb 2013 13:46:45 +0100] rev 51306
eliminated legacy 'axioms';
wenzelm [Thu, 28 Feb 2013 13:33:01 +0100] rev 51305
eliminated legacy 'axioms';
wenzelm [Thu, 28 Feb 2013 13:24:51 +0100] rev 51304
marginalized historic strip_tac;
wenzelm [Thu, 28 Feb 2013 13:19:25 +0100] rev 51303
tuned proof;
wenzelm [Thu, 28 Feb 2013 12:43:28 +0100] rev 51302
tuned whitespace and indentation;
wenzelm [Thu, 28 Feb 2013 12:24:24 +0100] rev 51301
simplified imports;
wenzelm [Thu, 28 Feb 2013 12:09:32 +0100] rev 51300
load timings in parallel for improved performance;
wenzelm [Thu, 28 Feb 2013 11:40:23 +0100] rev 51299
proper place for cancel_div_mod.ML (see also ee729dbd1b7f and ec7f10155389);
wenzelm [Wed, 27 Feb 2013 20:36:21 +0100] rev 51298
parallel dep.load_files saves approx. 1s on 4 cores;
wenzelm [Wed, 27 Feb 2013 19:39:16 +0100] rev 51297
eliminated pointless re-ified errors;
wenzelm [Wed, 27 Feb 2013 17:44:08 +0100] rev 51296
merged
wenzelm [Wed, 27 Feb 2013 17:32:17 +0100] rev 51295
discontinued redundant 'use' command;
wenzelm [Wed, 27 Feb 2013 16:27:44 +0100] rev 51294
discontinued obsolete header "files" -- these are loaded explicitly after exploring dependencies;
wenzelm [Wed, 27 Feb 2013 12:45:19 +0100] rev 51293
discontinued obsolete 'uses' within theory header;
Andreas Lochbihler [Wed, 27 Feb 2013 13:48:15 +0100] rev 51292
use lemma from Big_Operators
Andreas Lochbihler [Wed, 27 Feb 2013 13:44:19 +0100] rev 51291
add inclusion/exclusion lemma
Andreas Lochbihler [Wed, 27 Feb 2013 13:43:04 +0100] rev 51290
added lemma
Andreas Lochbihler [Wed, 27 Feb 2013 10:33:45 +0100] rev 51289
merged
Andreas Lochbihler [Wed, 27 Feb 2013 10:33:30 +0100] rev 51288
add wellorder instance for Numeral_Type (suggested by Jesus Aransay)
wenzelm [Tue, 26 Feb 2013 20:11:11 +0100] rev 51287
updated Toplevel.command_exception;
wenzelm [Tue, 26 Feb 2013 20:09:25 +0100] rev 51286
tuned;
wenzelm [Tue, 26 Feb 2013 19:58:27 +0100] rev 51285
tuned signature;
wenzelm [Tue, 26 Feb 2013 19:44:26 +0100] rev 51284
fork diagnostic commands (theory loader and PIDE interaction);
explicit id for load_thy, for more robust Goal.fork accounting and commit for each theory -- NB: use_thys nodes become subject to Position.is_reported like PIDE document transactions;
clarified Toplevel.command_exception vs. Toplevel.command_errors;
wenzelm [Tue, 26 Feb 2013 13:38:34 +0100] rev 51283
disallow shutdown from worker, which would lead to deadlock since the scheduler cannot terminate;
wenzelm [Tue, 26 Feb 2013 13:27:24 +0100] rev 51282
tuned 2464ba6e6fc9 -- NB: approximative_id is NONE for PIDE document transactions;
wenzelm [Tue, 26 Feb 2013 13:05:48 +0100] rev 51281
signal work_available should be sufficient to initiate daisy-chained workers, and lead to separate broadcast work_finished eventually -- NB: broadcasting all worker threads tends to burn parallel CPU cycles;
wenzelm [Tue, 26 Feb 2013 12:50:52 +0100] rev 51280
less eventful shutdown: merely wait for scheduler to terminate;
wenzelm [Tue, 26 Feb 2013 12:46:47 +0100] rev 51279
tuned messages;
wenzelm [Tue, 26 Feb 2013 11:57:19 +0100] rev 51278
tuned;
wenzelm [Mon, 25 Feb 2013 20:55:48 +0100] rev 51277
merged;
wenzelm [Mon, 25 Feb 2013 17:47:32 +0100] rev 51276
more explicit Goal.shutdown_futures;
wenzelm [Mon, 25 Feb 2013 13:31:02 +0100] rev 51275
reconsider 'export_code' as "thy_decl" command due to its global side-effect on the file-system;