Wed, 10 Nov 2010 18:15:21 -0800 move stuff from Domain.thy to Domain_Aux.thy
huffman [Wed, 10 Nov 2010 18:15:21 -0800] rev 40503
move stuff from Domain.thy to Domain_Aux.thy
Wed, 10 Nov 2010 17:56:08 -0800 move map functions to new theory file Map_Functions; add theory file Plain_HOLCF
huffman [Wed, 10 Nov 2010 17:56:08 -0800] rev 40502
move map functions to new theory file Map_Functions; add theory file Plain_HOLCF
Wed, 10 Nov 2010 14:59:52 -0800 allow unpointed lazy arguments for definitional domain package
huffman [Wed, 10 Nov 2010 14:59:52 -0800] rev 40501
allow unpointed lazy arguments for definitional domain package
Wed, 10 Nov 2010 14:20:47 -0800 add lemmas lub_below, below_lub; simplify some proofs; remove some unused lemmas
huffman [Wed, 10 Nov 2010 14:20:47 -0800] rev 40500
add lemmas lub_below, below_lub; simplify some proofs; remove some unused lemmas
Wed, 10 Nov 2010 13:22:39 -0800 merged
huffman [Wed, 10 Nov 2010 13:22:39 -0800] rev 40499
merged
Wed, 10 Nov 2010 13:08:42 -0800 removed unused lemma chain_mono2
huffman [Wed, 10 Nov 2010 13:08:42 -0800] rev 40498
removed unused lemma chain_mono2
Wed, 10 Nov 2010 11:42:35 -0800 rename class 'bifinite' to 'domain'
huffman [Wed, 10 Nov 2010 11:42:35 -0800] rev 40497
rename class 'bifinite' to 'domain'
Wed, 10 Nov 2010 09:59:08 -0800 instance sum :: (predomain, predomain) predomain
huffman [Wed, 10 Nov 2010 09:59:08 -0800] rev 40496
instance sum :: (predomain, predomain) predomain
Wed, 10 Nov 2010 09:52:50 -0800 configure sum type for fixrec
huffman [Wed, 10 Nov 2010 09:52:50 -0800] rev 40495
configure sum type for fixrec
Wed, 10 Nov 2010 08:18:32 -0800 add class liftdomain, for bifinite domains where DEFL('a u) = u_defl('a)
huffman [Wed, 10 Nov 2010 08:18:32 -0800] rev 40494
add class liftdomain, for bifinite domains where DEFL('a u) = u_defl('a)
Wed, 10 Nov 2010 06:02:37 -0800 instance prod :: (predomain, predomain) predomain
huffman [Wed, 10 Nov 2010 06:02:37 -0800] rev 40493
instance prod :: (predomain, predomain) predomain
Tue, 09 Nov 2010 19:37:11 -0800 adapt isodefl proof script to unpointed types
huffman [Tue, 09 Nov 2010 19:37:11 -0800] rev 40492
adapt isodefl proof script to unpointed types
Tue, 09 Nov 2010 16:37:13 -0800 add 'predomain' class: unpointed version of bifinite
huffman [Tue, 09 Nov 2010 16:37:13 -0800] rev 40491
add 'predomain' class: unpointed version of bifinite
Tue, 09 Nov 2010 08:41:36 -0800 add bifiniteness check for domain_isomorphism command
huffman [Tue, 09 Nov 2010 08:41:36 -0800] rev 40490
add bifiniteness check for domain_isomorphism command
Tue, 09 Nov 2010 05:23:34 -0800 implement map_of_typ using Pattern.rewrite_term
huffman [Tue, 09 Nov 2010 05:23:34 -0800] rev 40489
implement map_of_typ using Pattern.rewrite_term
Tue, 09 Nov 2010 04:47:46 -0800 avoid using stale theory
huffman [Tue, 09 Nov 2010 04:47:46 -0800] rev 40488
avoid using stale theory
Mon, 08 Nov 2010 15:13:45 -0800 implement defl_of_typ using Pattern.rewrite_term instead of DeflData theory data
huffman [Mon, 08 Nov 2010 15:13:45 -0800] rev 40487
implement defl_of_typ using Pattern.rewrite_term instead of DeflData theory data
Mon, 08 Nov 2010 14:36:17 -0800 add function the_sort
huffman [Mon, 08 Nov 2010 14:36:17 -0800] rev 40486
add function the_sort
Mon, 08 Nov 2010 14:09:07 -0800 refactor tmp_thy code
huffman [Mon, 08 Nov 2010 14:09:07 -0800] rev 40485
refactor tmp_thy code
Mon, 08 Nov 2010 06:58:09 -0800 reorganize Bifinite.thy; simplify some proofs related to bifinite class instances
huffman [Mon, 08 Nov 2010 06:58:09 -0800] rev 40484
reorganize Bifinite.thy; simplify some proofs related to bifinite class instances
Fri, 12 Nov 2010 11:36:01 +0100 treat pervasive "Interrupt" constructor as illegal -- superseded by Exn.Interrupt for internal use and Exn.is_interrupt/Exn.interrupt in user-space;
wenzelm [Fri, 12 Nov 2010 11:36:01 +0100] rev 40483
treat pervasive "Interrupt" constructor as illegal -- superseded by Exn.Interrupt for internal use and Exn.is_interrupt/Exn.interrupt in user-space;
Fri, 12 Nov 2010 10:58:09 +0100 Laze.force_result: more robust treatment of interrupts stemming from peer group cancellation;
wenzelm [Fri, 12 Nov 2010 10:58:09 +0100] rev 40482
Laze.force_result: more robust treatment of interrupts stemming from peer group cancellation;
Thu, 11 Nov 2010 19:58:07 +0100 more precise treatment of deleted nodes;
wenzelm [Thu, 11 Nov 2010 19:58:07 +0100] rev 40481
more precise treatment of deleted nodes;
Thu, 11 Nov 2010 18:55:17 +0100 tuned error message;
wenzelm [Thu, 11 Nov 2010 18:55:17 +0100] rev 40480
tuned error message;
Thu, 11 Nov 2010 17:07:05 +0100 unified type Document.Edit;
wenzelm [Thu, 11 Nov 2010 17:07:05 +0100] rev 40479
unified type Document.Edit;
Thu, 11 Nov 2010 16:48:46 +0100 replaced Document.Node_Text_Edit by Document.Text_Edit, with treatment of deleted nodes;
wenzelm [Thu, 11 Nov 2010 16:48:46 +0100] rev 40478
replaced Document.Node_Text_Edit by Document.Text_Edit, with treatment of deleted nodes; Document_Model.pending_edits: more robust treatment of init, including buffer reload event (jEdit 4.3.2 produces malformed remove/insert that lacks the last character); tuned;
Thu, 11 Nov 2010 13:23:39 +0100 tuned;
wenzelm [Thu, 11 Nov 2010 13:23:39 +0100] rev 40477
tuned;
Thu, 11 Nov 2010 13:07:41 +0100 reduced danger of line breaks within minipage;
wenzelm [Thu, 11 Nov 2010 13:07:41 +0100] rev 40476
reduced danger of line breaks within minipage;
Wed, 10 Nov 2010 20:43:22 +0100 Sidekick block asset: show first line only;
wenzelm [Wed, 10 Nov 2010 20:43:22 +0100] rev 40475
Sidekick block asset: show first line only;
Wed, 10 Nov 2010 20:21:55 +0100 added buffer_text convenience, with explicit locking;
wenzelm [Wed, 10 Nov 2010 20:21:55 +0100] rev 40474
added buffer_text convenience, with explicit locking;
Wed, 10 Nov 2010 17:53:41 +0100 use official/portable Multithreading.max_threads_value, which is also subject to user preferences (NB: Thread.numProcessors is apt to lead to surprises like very high numbers for systems with hyperthreading);
wenzelm [Wed, 10 Nov 2010 17:53:41 +0100] rev 40473
use official/portable Multithreading.max_threads_value, which is also subject to user preferences (NB: Thread.numProcessors is apt to lead to surprises like very high numbers for systems with hyperthreading);
Wed, 10 Nov 2010 16:05:15 +0100 merged
wenzelm [Wed, 10 Nov 2010 16:05:15 +0100] rev 40472
merged
Wed, 10 Nov 2010 09:03:07 +0100 make SML/NJ happy
blanchet [Wed, 10 Nov 2010 09:03:07 +0100] rev 40471
make SML/NJ happy
Tue, 09 Nov 2010 16:18:40 +0100 merged
haftmann [Tue, 09 Nov 2010 16:18:40 +0100] rev 40470
merged
Tue, 09 Nov 2010 14:02:14 +0100 slightly changed fun_map_def
haftmann [Tue, 09 Nov 2010 14:02:14 +0100] rev 40469
slightly changed fun_map_def
Tue, 09 Nov 2010 14:02:14 +0100 fun_rel_def is no simp rule by default
haftmann [Tue, 09 Nov 2010 14:02:14 +0100] rev 40468
fun_rel_def is no simp rule by default
Tue, 09 Nov 2010 14:02:13 +0100 more appropriate specification packages; fun_rel_def is no simp rule by default
haftmann [Tue, 09 Nov 2010 14:02:13 +0100] rev 40467
more appropriate specification packages; fun_rel_def is no simp rule by default
Tue, 09 Nov 2010 14:02:13 +0100 type annotations in specifications; fun_rel_def is no simp rule by default; slightly changed fun_map_def; more on predicates on relation functions; proper HOL equations in definitions
haftmann [Tue, 09 Nov 2010 14:02:13 +0100] rev 40466
type annotations in specifications; fun_rel_def is no simp rule by default; slightly changed fun_map_def; more on predicates on relation functions; proper HOL equations in definitions
Tue, 09 Nov 2010 14:02:13 +0100 more appropriate specification packages; fun_rel_def is no simp rule by default
haftmann [Tue, 09 Nov 2010 14:02:13 +0100] rev 40465
more appropriate specification packages; fun_rel_def is no simp rule by default
Tue, 09 Nov 2010 14:02:12 +0100 type annotations in specifications; fun_rel_def is no simp rule by default
haftmann [Tue, 09 Nov 2010 14:02:12 +0100] rev 40464
type annotations in specifications; fun_rel_def is no simp rule by default
Tue, 09 Nov 2010 14:02:12 +0100 fun_rel_def is no simp rule by default
haftmann [Tue, 09 Nov 2010 14:02:12 +0100] rev 40463
fun_rel_def is no simp rule by default
Tue, 09 Nov 2010 14:00:10 +0000 merged
paulson [Tue, 09 Nov 2010 14:00:10 +0000] rev 40462
merged
Tue, 09 Nov 2010 13:59:37 +0000 tidied using metis
paulson [Tue, 09 Nov 2010 13:59:37 +0000] rev 40461
tidied using metis
Wed, 10 Nov 2010 15:59:23 +0100 manage folding via sidekick by default;
wenzelm [Wed, 10 Nov 2010 15:59:23 +0100] rev 40460
manage folding via sidekick by default;
Wed, 10 Nov 2010 15:47:56 +0100 eliminated obsolete heading category -- superseded by heading_level;
wenzelm [Wed, 10 Nov 2010 15:47:56 +0100] rev 40459
eliminated obsolete heading category -- superseded by heading_level;
Wed, 10 Nov 2010 15:43:06 +0100 treat main theory commands like headings, and nest anything else inside;
wenzelm [Wed, 10 Nov 2010 15:43:06 +0100] rev 40458
treat main theory commands like headings, and nest anything else inside;
Wed, 10 Nov 2010 15:42:20 +0100 proper treatment of equal heading level;
wenzelm [Wed, 10 Nov 2010 15:42:20 +0100] rev 40457
proper treatment of equal heading level;
Wed, 10 Nov 2010 15:41:29 +0100 added missing Keyword.THY_SCHEMATIC_GOAL;
wenzelm [Wed, 10 Nov 2010 15:41:29 +0100] rev 40456
added missing Keyword.THY_SCHEMATIC_GOAL; more keyword categories;
Wed, 10 Nov 2010 15:17:25 +0100 default Sidekick parser based on section headings;
wenzelm [Wed, 10 Nov 2010 15:17:25 +0100] rev 40455
default Sidekick parser based on section headings;
Wed, 10 Nov 2010 15:00:40 +0100 some support for nested source structure, based on section headings;
wenzelm [Wed, 10 Nov 2010 15:00:40 +0100] rev 40454
some support for nested source structure, based on section headings;
Wed, 10 Nov 2010 11:44:35 +0100 tuned;
wenzelm [Wed, 10 Nov 2010 11:44:35 +0100] rev 40453
tuned;
Tue, 09 Nov 2010 23:24:46 +0100 misc tuning and simplification, using Isabelle_Sidekick.Asset (not sidekick.Asset, which is dynamically dispatched to slightly different semantics);
wenzelm [Tue, 09 Nov 2010 23:24:46 +0100] rev 40452
misc tuning and simplification, using Isabelle_Sidekick.Asset (not sidekick.Asset, which is dynamically dispatched to slightly different semantics);
Tue, 09 Nov 2010 22:37:10 +0100 updated version;
wenzelm [Tue, 09 Nov 2010 22:37:10 +0100] rev 40451
updated version;
Tue, 09 Nov 2010 21:52:05 +0100 private counter, to keep externalized ids a bit smaller;
wenzelm [Tue, 09 Nov 2010 21:52:05 +0100] rev 40450
private counter, to keep externalized ids a bit smaller;
Tue, 09 Nov 2010 21:44:19 +0100 added general Synchronized.counter convenience;
wenzelm [Tue, 09 Nov 2010 21:44:19 +0100] rev 40449
added general Synchronized.counter convenience;
Tue, 09 Nov 2010 21:13:06 +0100 explicitly identify forked/joined tasks;
wenzelm [Tue, 09 Nov 2010 21:13:06 +0100] rev 40448
explicitly identify forked/joined tasks;
Tue, 09 Nov 2010 11:27:58 +0100 accomodate old manuals that include pdfsetup.sty without isabelle.sty;
wenzelm [Tue, 09 Nov 2010 11:27:58 +0100] rev 40447
accomodate old manuals that include pdfsetup.sty without isabelle.sty;
Tue, 09 Nov 2010 11:17:15 +0100 merged
wenzelm [Tue, 09 Nov 2010 11:17:15 +0100] rev 40446
merged
Mon, 08 Nov 2010 23:02:20 +0100 removed type-inference-like behaviour from relation_tac completely; tuned
krauss [Mon, 08 Nov 2010 23:02:20 +0100] rev 40445
removed type-inference-like behaviour from relation_tac completely; tuned
Mon, 08 Nov 2010 20:55:27 +0100 avoid clash of \<upharpoonright> vs. \<restriction> (cf. 666ea7e62384 and 3c49dbece0a8);
wenzelm [Mon, 08 Nov 2010 20:55:27 +0100] rev 40444
avoid clash of \<upharpoonright> vs. \<restriction> (cf. 666ea7e62384 and 3c49dbece0a8);
Mon, 08 Nov 2010 20:50:56 +0100 explicitly check uniqueness of symbol recoding;
wenzelm [Mon, 08 Nov 2010 20:50:56 +0100] rev 40443
explicitly check uniqueness of symbol recoding;
Mon, 08 Nov 2010 17:44:47 +0100 more hints on building and running Isabelle/jEdit from command line;
wenzelm [Mon, 08 Nov 2010 17:44:47 +0100] rev 40442
more hints on building and running Isabelle/jEdit from command line;
Mon, 08 Nov 2010 14:41:11 +0100 merged
wenzelm [Mon, 08 Nov 2010 14:41:11 +0100] rev 40441
merged
Mon, 08 Nov 2010 14:33:54 +0100 merge
blanchet [Mon, 08 Nov 2010 14:33:54 +0100] rev 40440
merge
Mon, 08 Nov 2010 14:33:30 +0100 reduce the number of monomorphization iterations from 10 (the default) to 4, in the interest of faster SMT solving
blanchet [Mon, 08 Nov 2010 14:33:30 +0100] rev 40439
reduce the number of monomorphization iterations from 10 (the default) to 4, in the interest of faster SMT solving
Mon, 08 Nov 2010 05:07:18 -0800 merged
huffman [Mon, 08 Nov 2010 05:07:18 -0800] rev 40438
merged
Sat, 06 Nov 2010 10:01:00 -0700 merged
huffman [Sat, 06 Nov 2010 10:01:00 -0700] rev 40437
merged
Fri, 05 Nov 2010 15:15:28 -0700 (infixl "<<" 55) -> (infix "<<" 50)
huffman [Fri, 05 Nov 2010 15:15:28 -0700] rev 40436
(infixl "<<" 55) -> (infix "<<" 50)
Wed, 03 Nov 2010 17:22:25 -0700 simplify some proofs
huffman [Wed, 03 Nov 2010 17:22:25 -0700] rev 40435
simplify some proofs
Wed, 03 Nov 2010 17:06:21 -0700 remove unnecessary stuff from Discrete.thy
huffman [Wed, 03 Nov 2010 17:06:21 -0700] rev 40434
remove unnecessary stuff from Discrete.thy
Wed, 03 Nov 2010 16:39:23 -0700 remove some unnecessary lemmas; move monofun_LAM to Cfun.thy
huffman [Wed, 03 Nov 2010 16:39:23 -0700] rev 40433
remove some unnecessary lemmas; move monofun_LAM to Cfun.thy
Wed, 03 Nov 2010 15:57:39 -0700 add lemma eq_imp_below
huffman [Wed, 03 Nov 2010 15:57:39 -0700] rev 40432
add lemma eq_imp_below
Wed, 03 Nov 2010 15:47:46 -0700 discontinue a bunch of legacy theorem names
huffman [Wed, 03 Nov 2010 15:47:46 -0700] rev 40431
discontinue a bunch of legacy theorem names
Wed, 03 Nov 2010 15:31:24 -0700 move a few admissibility lemmas into FOCUS/Stream_adm.thy
huffman [Wed, 03 Nov 2010 15:31:24 -0700] rev 40430
move a few admissibility lemmas into FOCUS/Stream_adm.thy
Wed, 03 Nov 2010 15:03:16 -0700 simplify some proofs
huffman [Wed, 03 Nov 2010 15:03:16 -0700] rev 40429
simplify some proofs
Mon, 08 Nov 2010 13:53:18 +0100 compile -- 7550b2cba1cb broke the build
blanchet [Mon, 08 Nov 2010 13:53:18 +0100] rev 40428
compile -- 7550b2cba1cb broke the build
Mon, 08 Nov 2010 13:25:00 +0100 merge
blanchet [Mon, 08 Nov 2010 13:25:00 +0100] rev 40427
merge
Mon, 08 Nov 2010 09:10:44 +0100 recognize Vampire error
blanchet [Mon, 08 Nov 2010 09:10:44 +0100] rev 40426
recognize Vampire error
Mon, 08 Nov 2010 12:13:51 +0100 return the process return code along with the process outputs
boehmes [Mon, 08 Nov 2010 12:13:51 +0100] rev 40425
return the process return code along with the process outputs
Mon, 08 Nov 2010 12:13:44 +0100 better modularization: moved SMT configuration options and diagnostics as well as SMT failure and exception into separate structures (both of which are loaded first and consequently are available to other SMT structures)
boehmes [Mon, 08 Nov 2010 12:13:44 +0100] rev 40424
better modularization: moved SMT configuration options and diagnostics as well as SMT failure and exception into separate structures (both of which are loaded first and consequently are available to other SMT structures)
Mon, 08 Nov 2010 11:49:28 +0100 merged
haftmann [Mon, 08 Nov 2010 11:49:28 +0100] rev 40423
merged
Mon, 08 Nov 2010 10:56:48 +0100 corrected slip: must keep constant map, not type map; tuned code
haftmann [Mon, 08 Nov 2010 10:56:48 +0100] rev 40422
corrected slip: must keep constant map, not type map; tuned code
Mon, 08 Nov 2010 10:43:24 +0100 constructors to datatypes in code_reflect can be globbed; dropped unused code
haftmann [Mon, 08 Nov 2010 10:43:24 +0100] rev 40421
constructors to datatypes in code_reflect can be globbed; dropped unused code
Mon, 08 Nov 2010 09:25:43 +0100 adding code and theory for smallvalue generators, but do not setup the interpretation yet
bulwahn [Mon, 08 Nov 2010 09:25:43 +0100] rev 40420
adding code and theory for smallvalue generators, but do not setup the interpretation yet
Mon, 08 Nov 2010 02:33:48 +0100 make sure the SMT solver runs several iterations by lowering the timeout at each iteration -- yields better results in practice
blanchet [Mon, 08 Nov 2010 02:33:48 +0100] rev 40419
make sure the SMT solver runs several iterations by lowering the timeout at each iteration -- yields better results in practice
Mon, 08 Nov 2010 02:32:27 +0100 better detection of completely irrelevant facts
blanchet [Mon, 08 Nov 2010 02:32:27 +0100] rev 40418
better detection of completely irrelevant facts
Sun, 07 Nov 2010 18:19:04 +0100 always use a hard timeout in Mirabelle
blanchet [Sun, 07 Nov 2010 18:19:04 +0100] rev 40417
always use a hard timeout in Mirabelle
Sun, 07 Nov 2010 18:15:13 +0100 use "smt" (rather than "metis") to reconstruct SMT proofs
blanchet [Sun, 07 Nov 2010 18:15:13 +0100] rev 40416
use "smt" (rather than "metis") to reconstruct SMT proofs
Sun, 07 Nov 2010 18:03:24 +0100 don't pass too many facts on the first iteration of the SMT solver
blanchet [Sun, 07 Nov 2010 18:03:24 +0100] rev 40415
don't pass too many facts on the first iteration of the SMT solver
Sun, 07 Nov 2010 18:02:02 +0100 catch TimeOut exception
blanchet [Sun, 07 Nov 2010 18:02:02 +0100] rev 40414
catch TimeOut exception
Sun, 07 Nov 2010 17:56:07 +0100 ensure the SMT solver respects the timeout -- Mirabelle revealed cases where "smt_filter" apparently never returns
blanchet [Sun, 07 Nov 2010 17:56:07 +0100] rev 40413
ensure the SMT solver respects the timeout -- Mirabelle revealed cases where "smt_filter" apparently never returns
Sun, 07 Nov 2010 17:51:25 +0100 if SMT used as a filter in a loop fails at each iteration, returns the first error, not the last, since it is more informative -- the first error typically says "out of memory", whereas the last might well be "the SMT problem is unprovable", which should be no surprise if too many facts were removed
blanchet [Sun, 07 Nov 2010 17:51:25 +0100] rev 40412
if SMT used as a filter in a loop fails at each iteration, returns the first error, not the last, since it is more informative -- the first error typically says "out of memory", whereas the last might well be "the SMT problem is unprovable", which should be no surprise if too many facts were removed
Sun, 07 Nov 2010 13:29:59 +0100 removed explicit "Interrupt" handling for conformity with async model -- unfortunately the user loses the information about how many scopes were checked, but this needs to be retought with the new interface anyway
blanchet [Sun, 07 Nov 2010 13:29:59 +0100] rev 40411
removed explicit "Interrupt" handling for conformity with async model -- unfortunately the user loses the information about how many scopes were checked, but this needs to be retought with the new interface anyway
Sat, 06 Nov 2010 10:25:08 +0100 make Nitpick datatype tests faster to make timeout less likely
blanchet [Sat, 06 Nov 2010 10:25:08 +0100] rev 40410
make Nitpick datatype tests faster to make timeout less likely
Sat, 06 Nov 2010 10:25:08 +0100 invoke SMT solver in a loop, with fewer and fewer facts, in case of error
blanchet [Sat, 06 Nov 2010 10:25:08 +0100] rev 40409
invoke SMT solver in a loop, with fewer and fewer facts, in case of error
Sat, 06 Nov 2010 10:25:08 +0100 always honor the max relevant constraint
blanchet [Sat, 06 Nov 2010 10:25:08 +0100] rev 40408
always honor the max relevant constraint
(0) -30000 -10000 -3000 -1000 -300 -100 -96 +96 +100 +300 +1000 +3000 +10000 +30000 tip