krauss [Fri, 06 Nov 2009 13:49:19 +0100] rev 33470
NEWS
krauss [Fri, 06 Nov 2009 13:42:29 +0100] rev 33469
removed session SizeChange: outdated, only half-functional, alternatives exist (cf. size_change method)
krauss [Fri, 06 Nov 2009 13:36:46 +0100] rev 33468
renamed method sizechange to size_change
krauss [Fri, 06 Nov 2009 12:13:45 +0100] rev 33467
added boehmes and hoelzl to isatest mailings
wenzelm [Fri, 06 Nov 2009 10:26:13 +0100] rev 33466
merged
boehmes [Fri, 06 Nov 2009 09:27:20 +0100] rev 33465
tuned
ballarin [Thu, 05 Nov 2009 20:42:47 +0100] rev 33464
Merged.
ballarin [Wed, 04 Nov 2009 22:54:42 +0100] rev 33463
Merged.
ballarin [Wed, 04 Nov 2009 22:51:27 +0100] rev 33462
Use PrintMode.setmp to make thread-safe; avoid code clones.
ballarin [Mon, 02 Nov 2009 22:51:22 +0100] rev 33461
Make output indenpendent of current print mode.
ballarin [Mon, 02 Nov 2009 21:27:26 +0100] rev 33460
Relax on type agreement with original context when applying term syntax.
wenzelm [Thu, 05 Nov 2009 23:59:23 +0100] rev 33459
tuned;
wenzelm [Thu, 05 Nov 2009 22:59:57 +0100] rev 33458
proper naming convention lthy: local_theory, but ctxt: Proof.context for arbitrary context;
tuned signature;
tuned;
wenzelm [Thu, 05 Nov 2009 22:08:47 +0100] rev 33457
adapted LocalTheory.declaration;
wenzelm [Thu, 05 Nov 2009 22:06:46 +0100] rev 33456
allow "pervasive" local theory declarations, which are applied the background theory;
wenzelm [Thu, 05 Nov 2009 20:44:42 +0100] rev 33455
declare Spec_Rules for most basic definitional packages;
wenzelm [Thu, 05 Nov 2009 20:41:45 +0100] rev 33454
misc tuning and clarification;
wenzelm [Thu, 05 Nov 2009 20:40:16 +0100] rev 33453
scalable version of Named_Thms, using Item_Net;
wenzelm [Thu, 05 Nov 2009 17:59:49 +0100] rev 33452
merged
wenzelm [Thu, 05 Nov 2009 17:36:15 +0100] rev 33451
merged
wenzelm [Thu, 05 Nov 2009 16:23:51 +0100] rev 33450
more accurate cleanup;
wenzelm [Thu, 05 Nov 2009 15:55:07 +0100] rev 33449
merged
wenzelm [Thu, 05 Nov 2009 15:54:14 +0100] rev 33448
more accurate dependencies;
boehmes [Thu, 05 Nov 2009 15:44:39 +0100] rev 33447
merged
boehmes [Thu, 05 Nov 2009 15:24:49 +0100] rev 33446
handle let expressions inside terms by unfolding (instead of raising an exception),
added examples to test this feature
boehmes [Thu, 05 Nov 2009 14:48:40 +0100] rev 33445
shorter names for variables and verification conditions,
auto-fix variables occurring in a verification condition
boehmes [Thu, 05 Nov 2009 14:41:37 +0100] rev 33444
added references to HOL-Boogie papers
wenzelm [Thu, 05 Nov 2009 17:58:58 +0100] rev 33443
tuned header;
use plain simultaneous lemma statements -- Pure's &&& should hardly ever occur in user space;
wenzelm [Thu, 05 Nov 2009 17:02:43 +0100] rev 33442
made SML/NJ happy;
normalized type abbreviations;
wenzelm [Thu, 05 Nov 2009 16:10:49 +0100] rev 33441
eliminated funny record patterns and made SML/NJ happy;
wenzelm [Thu, 05 Nov 2009 14:47:27 +0100] rev 33440
proper header;
eliminated SML97's opaque signature constrain, which is essentially a legacy feature (due to problems with ML toplevel pretty printing);
wenzelm [Thu, 05 Nov 2009 14:37:39 +0100] rev 33439
more accurate dependencies;
tuned;
wenzelm [Thu, 05 Nov 2009 13:57:56 +0100] rev 33438
merged
krauss [Wed, 04 Nov 2009 17:17:30 +0100] rev 33437
added Tree23 to IsaMakefile
nipkow [Wed, 04 Nov 2009 16:54:22 +0100] rev 33436
New
nipkow [Wed, 04 Nov 2009 10:17:58 +0100] rev 33435
merged
nipkow [Wed, 04 Nov 2009 10:17:43 +0100] rev 33434
fixed order of parameters in induction rules
krauss [Wed, 04 Nov 2009 09:43:25 +0100] rev 33433
added bulwahn to isatest mailings
nipkow [Wed, 04 Nov 2009 09:18:46 +0100] rev 33432
merged
nipkow [Wed, 04 Nov 2009 09:18:03 +0100] rev 33431
Completely overhauled
huffman [Tue, 03 Nov 2009 19:01:06 -0800] rev 33430
better error handling for fixrec_simp
huffman [Tue, 03 Nov 2009 18:33:16 -0800] rev 33429
add more fixrec_simp rules
huffman [Tue, 03 Nov 2009 18:32:56 -0800] rev 33428
fixrec examples use fixrec_simp instead of fixpat
huffman [Tue, 03 Nov 2009 18:32:30 -0800] rev 33427
domain package registers fixrec_simp lemmas
huffman [Tue, 03 Nov 2009 17:09:27 -0800] rev 33426
merged
huffman [Tue, 03 Nov 2009 17:03:21 -0800] rev 33425
add fixrec_simp attribute and method (eventually to replace fixpat)
boehmes [Tue, 03 Nov 2009 23:44:16 +0100] rev 33424
proper and unique case names for the split_vc method,
shortened label names,
added an example demonstrating the split_vc method
haftmann [Tue, 03 Nov 2009 19:32:08 +0100] rev 33423
merged
haftmann [Tue, 03 Nov 2009 17:08:57 +0100] rev 33422
merged
haftmann [Tue, 03 Nov 2009 17:06:35 +0100] rev 33421
always be qualified -- suspected smartness in fact never worked as expected
haftmann [Tue, 03 Nov 2009 17:06:08 +0100] rev 33420
pretty name for ==>
boehmes [Tue, 03 Nov 2009 17:54:24 +0100] rev 33419
added HOL-Boogie
boehmes [Tue, 03 Nov 2009 14:51:55 +0100] rev 33418
added a specific SMT exception captured by smt_tac (prevents the SMT method from failing with an exception),
replaced unspecific 'error' invocations with raising of specific SMT exceptions,
added annotations to traced SMT problem and solver output
boehmes [Tue, 03 Nov 2009 14:07:38 +0100] rev 33417
ignore parsing errors, return empty assignment instead
wenzelm [Thu, 05 Nov 2009 13:16:22 +0100] rev 33416
scheduler: clarified interrupt attributes and handling;
wenzelm [Thu, 05 Nov 2009 13:01:11 +0100] rev 33415
worker_next: plain signalling via work_available only, not scheduler_event;
scheduler: tuned worker pool adjustments;
wenzelm [Thu, 05 Nov 2009 00:13:00 +0100] rev 33414
revert fulfill_proof_future tuning (actually a bit slower due to granularity issues?);
wenzelm [Wed, 04 Nov 2009 21:22:35 +0100] rev 33413
avoid broadcast work_available, use daisy-chained signal instead;
max_threads: allow as much as 4 * m, after extra delay;
wenzelm [Wed, 04 Nov 2009 21:21:05 +0100] rev 33412
fulfill_proof_future: tuned important special case of singleton promise;
wenzelm [Wed, 04 Nov 2009 20:31:36 +0100] rev 33411
worker_next: treat wait for work_available as Sleeping, not Waiting;
max_threads: simple adaptive scheme between m and 2 * m;