Sat, 15 Feb 2014 18:48:43 +0100 removed dead code;
wenzelm [Sat, 15 Feb 2014 18:48:43 +0100] rev 55506
removed dead code; tuned;
Sat, 15 Feb 2014 18:28:18 +0100 more uniform ML keyword markup;
wenzelm [Sat, 15 Feb 2014 18:28:18 +0100] rev 55505
more uniform ML keyword markup; tuned;
Sat, 15 Feb 2014 17:10:57 +0100 merged
wenzelm [Sat, 15 Feb 2014 17:10:57 +0100] rev 55504
merged
Sat, 15 Feb 2014 17:04:55 +0100 tuned;
wenzelm [Sat, 15 Feb 2014 17:04:55 +0100] rev 55503
tuned;
Sat, 15 Feb 2014 16:55:48 +0100 clarified Isabelle/ML strings;
wenzelm [Sat, 15 Feb 2014 16:55:48 +0100] rev 55502
clarified Isabelle/ML strings;
Sat, 15 Feb 2014 16:49:10 +0100 refined ML keyword styles;
wenzelm [Sat, 15 Feb 2014 16:49:10 +0100] rev 55501
refined ML keyword styles;
Sat, 15 Feb 2014 16:27:58 +0100 isabelle-ml mode with separate token marker;
wenzelm [Sat, 15 Feb 2014 16:27:58 +0100] rev 55500
isabelle-ml mode with separate token marker; clarified ML_Lex.gap_start: end-of-input counts as single newline;
Sat, 15 Feb 2014 14:52:51 +0100 partial scans via ML_Lex.tokenize_context;
wenzelm [Sat, 15 Feb 2014 14:52:51 +0100] rev 55499
partial scans via ML_Lex.tokenize_context; simplified ML_char: no gaps (hardly relevant in practice); tuned;
Fri, 14 Feb 2014 22:03:48 +0100 proper signature;
wenzelm [Fri, 14 Feb 2014 22:03:48 +0100] rev 55498
proper signature; removed dead code;
Fri, 14 Feb 2014 21:06:20 +0100 lexical syntax for SML (in Scala);
wenzelm [Fri, 14 Feb 2014 21:06:20 +0100] rev 55497
lexical syntax for SML (in Scala); tuned;
Fri, 14 Feb 2014 20:58:48 +0100 tuned;
wenzelm [Fri, 14 Feb 2014 20:58:48 +0100] rev 55496
tuned;
Fri, 14 Feb 2014 16:27:29 +0100 removed dead code;
wenzelm [Fri, 14 Feb 2014 16:27:29 +0100] rev 55495
removed dead code;
Fri, 14 Feb 2014 16:25:30 +0100 tuned signature (in accordance to ML version);
wenzelm [Fri, 14 Feb 2014 16:25:30 +0100] rev 55494
tuned signature (in accordance to ML version);
Fri, 14 Feb 2014 16:11:14 +0100 tuned proofs;
wenzelm [Fri, 14 Feb 2014 16:11:14 +0100] rev 55493
tuned proofs;
Fri, 14 Feb 2014 15:42:27 +0100 tuned signature -- separate Lexicon from Parsers (in accordance to ML version);
wenzelm [Fri, 14 Feb 2014 15:42:27 +0100] rev 55492
tuned signature -- separate Lexicon from Parsers (in accordance to ML version);
Fri, 14 Feb 2014 14:52:50 +0100 prefer latest ProofGeneral-4.2-1 by default;
wenzelm [Fri, 14 Feb 2014 14:52:50 +0100] rev 55491
prefer latest ProofGeneral-4.2-1 by default;
Fri, 14 Feb 2014 14:51:38 +0100 updated thy_info.dependencies;
wenzelm [Fri, 14 Feb 2014 14:51:38 +0100] rev 55490
updated thy_info.dependencies;
Fri, 14 Feb 2014 14:44:43 +0100 tuned message;
wenzelm [Fri, 14 Feb 2014 14:44:43 +0100] rev 55489
tuned message;
Fri, 14 Feb 2014 14:39:44 +0100 more integrity checks of theory names vs. full node names;
wenzelm [Fri, 14 Feb 2014 14:39:44 +0100] rev 55488
more integrity checks of theory names vs. full node names;
Sat, 15 Feb 2014 00:11:17 +0100 abstract type must be a type constructor; check it
kuncar [Sat, 15 Feb 2014 00:11:17 +0100] rev 55487
abstract type must be a type constructor; check it
Fri, 14 Feb 2014 18:42:43 +0100 generate proper 'DtRec' indices in 'datatype_new_compat' for the case where some types are duplicated
blanchet [Fri, 14 Feb 2014 18:42:43 +0100] rev 55486
generate proper 'DtRec' indices in 'datatype_new_compat' for the case where some types are duplicated
Fri, 14 Feb 2014 17:18:28 +0100 better handling of recursion through functions
blanchet [Fri, 14 Feb 2014 17:18:28 +0100] rev 55485
better handling of recursion through functions
Fri, 14 Feb 2014 16:22:09 +0100 added examples/tests
blanchet [Fri, 14 Feb 2014 16:22:09 +0100] rev 55484
added examples/tests
Fri, 14 Feb 2014 16:21:41 +0100 tuned code to allow mutualized corecursion through different functions with the same target type
blanchet [Fri, 14 Feb 2014 16:21:41 +0100] rev 55483
tuned code to allow mutualized corecursion through different functions with the same target type
Fri, 14 Feb 2014 15:39:43 +0100 removed assumption in 'primrec_new' that a given constructor can only occur once
blanchet [Fri, 14 Feb 2014 15:39:43 +0100] rev 55482
removed assumption in 'primrec_new' that a given constructor can only occur once
Fri, 14 Feb 2014 15:14:35 +0100 generate unique names
blanchet [Fri, 14 Feb 2014 15:14:35 +0100] rev 55481
generate unique names
Fri, 14 Feb 2014 15:03:24 +0100 allow different functions to recurse on the same type, like in the old package
blanchet [Fri, 14 Feb 2014 15:03:24 +0100] rev 55480
allow different functions to recurse on the same type, like in the old package
Fri, 14 Feb 2014 15:03:23 +0100 improved 'datatype_new_compat': generate more fixpoint equations for types like 'datatype_new x = C (x list) (x list)' (here, one equation for each x list instead of a single for both), for higher compatibility + code generation attributes on the recursor
blanchet [Fri, 14 Feb 2014 15:03:23 +0100] rev 55479
improved 'datatype_new_compat': generate more fixpoint equations for types like 'datatype_new x = C (x list) (x list)' (here, one equation for each x list instead of a single for both), for higher compatibility + code generation attributes on the recursor
Fri, 14 Feb 2014 14:54:08 +0100 made N2M more robust w.r.t. identical nested types
traytel [Fri, 14 Feb 2014 14:54:08 +0100] rev 55478
made N2M more robust w.r.t. identical nested types
Fri, 14 Feb 2014 13:45:29 +0100 register bnfs for (co)datatypes under their proper name (lost in af71b753c459)
traytel [Fri, 14 Feb 2014 13:45:29 +0100] rev 55477
register bnfs for (co)datatypes under their proper name (lost in af71b753c459)
Fri, 14 Feb 2014 11:10:28 +0100 updated keywords;
wenzelm [Fri, 14 Feb 2014 11:10:28 +0100] rev 55476
updated keywords;
Fri, 14 Feb 2014 10:33:57 +0100 restored old 'remotify' logic -- too many bugs were introduced when refactoring the code
blanchet [Fri, 14 Feb 2014 10:33:57 +0100] rev 55475
restored old 'remotify' logic -- too many bugs were introduced when refactoring the code
Fri, 14 Feb 2014 07:53:46 +0100 more (co)datatype docs
blanchet [Fri, 14 Feb 2014 07:53:46 +0100] rev 55474
more (co)datatype docs
Fri, 14 Feb 2014 07:53:46 +0100 hide 'rel' name -- this one is waiting to be merged with 'list_all2'
blanchet [Fri, 14 Feb 2014 07:53:46 +0100] rev 55473
hide 'rel' name -- this one is waiting to be merged with 'list_all2'
Fri, 14 Feb 2014 07:53:46 +0100 updated docs to reflect the new 'free_constructors' syntax
blanchet [Fri, 14 Feb 2014 07:53:46 +0100] rev 55472
updated docs to reflect the new 'free_constructors' syntax
Fri, 14 Feb 2014 07:53:46 +0100 more precise spec rules for selectors
blanchet [Fri, 14 Feb 2014 07:53:46 +0100] rev 55471
more precise spec rules for selectors
Fri, 14 Feb 2014 07:53:46 +0100 removed needless robustness (no longer needed thanks to new syntax)
blanchet [Fri, 14 Feb 2014 07:53:46 +0100] rev 55470
removed needless robustness (no longer needed thanks to new syntax)
Fri, 14 Feb 2014 07:53:46 +0100 aligned the syntax for 'free_constructors' on the 'datatype_new' and 'codatatype' syntax
blanchet [Fri, 14 Feb 2014 07:53:46 +0100] rev 55469
aligned the syntax for 'free_constructors' on the 'datatype_new' and 'codatatype' syntax
Fri, 14 Feb 2014 07:53:46 +0100 renamed 'wrap_free_constructors' to 'free_constructors' (cf. 'functor', 'bnf', etc.)
blanchet [Fri, 14 Feb 2014 07:53:46 +0100] rev 55468
renamed 'wrap_free_constructors' to 'free_constructors' (cf. 'functor', 'bnf', etc.)
Fri, 14 Feb 2014 07:53:46 +0100 renamed 'enriched_type' to more informative 'functor' (following the renaming of enriched type constructors to bounded natural functors)
blanchet [Fri, 14 Feb 2014 07:53:46 +0100] rev 55467
renamed 'enriched_type' to more informative 'functor' (following the renaming of enriched type constructors to bounded natural functors)
Fri, 14 Feb 2014 07:53:46 +0100 merged 'Option.map' and 'Option.map_option'
blanchet [Fri, 14 Feb 2014 07:53:46 +0100] rev 55466
merged 'Option.map' and 'Option.map_option'
Fri, 14 Feb 2014 07:53:45 +0100 merged 'List.map' and 'List.list.map'
blanchet [Fri, 14 Feb 2014 07:53:45 +0100] rev 55465
merged 'List.map' and 'List.list.map'
Fri, 14 Feb 2014 07:53:45 +0100 have 'Ctr_Sugar' register its 'Spec_Rules'
blanchet [Fri, 14 Feb 2014 07:53:45 +0100] rev 55464
have 'Ctr_Sugar' register its 'Spec_Rules'
Fri, 14 Feb 2014 07:53:45 +0100 register 'Spec_Rules' for new-style (co)datatypes
blanchet [Fri, 14 Feb 2014 07:53:45 +0100] rev 55463
register 'Spec_Rules' for new-style (co)datatypes
Fri, 14 Feb 2014 07:53:45 +0100 added 'Spec_Rules' for 'primcorec'
blanchet [Fri, 14 Feb 2014 07:53:45 +0100] rev 55462
added 'Spec_Rules' for 'primcorec'
Thu, 13 Feb 2014 22:35:38 +0100 more integrity checks of theory names vs. full node names -- at least for the scope of a single use_thys (or "theories" section in ROOT);
wenzelm [Thu, 13 Feb 2014 22:35:38 +0100] rev 55461
more integrity checks of theory names vs. full node names -- at least for the scope of a single use_thys (or "theories" section in ROOT);
Thu, 13 Feb 2014 17:11:25 +0100 added a bit of documentation for the different commands
blanchet [Thu, 13 Feb 2014 17:11:25 +0100] rev 55460
added a bit of documentation for the different commands
Thu, 13 Feb 2014 17:11:11 +0100 cleaner, complete proof in documentation, contributed by Dmitriy T.
blanchet [Thu, 13 Feb 2014 17:11:11 +0100] rev 55459
cleaner, complete proof in documentation, contributed by Dmitriy T.
Thu, 13 Feb 2014 16:21:43 +0100 do the right thing with provers that exist only remotely (e.g. e_sine)
blanchet [Thu, 13 Feb 2014 16:21:43 +0100] rev 55458
do the right thing with provers that exist only remotely (e.g. e_sine)
Thu, 13 Feb 2014 15:51:54 +0100 more precise descripiton
kuncar [Thu, 13 Feb 2014 15:51:54 +0100] rev 55457
more precise descripiton
Thu, 13 Feb 2014 14:32:05 +0100 all_args_conv works also for zero arguments
kuncar [Thu, 13 Feb 2014 14:32:05 +0100] rev 55456
all_args_conv works also for zero arguments
Thu, 13 Feb 2014 14:32:04 +0100 don't catch QOUT_THM_INTERNAL from the recursive call of parametrize_relation_conv
kuncar [Thu, 13 Feb 2014 14:32:04 +0100] rev 55455
don't catch QOUT_THM_INTERNAL from the recursive call of parametrize_relation_conv
Wed, 12 Feb 2014 18:32:55 +0100 Lifting: support a type variable as a raw type
kuncar [Wed, 12 Feb 2014 18:32:55 +0100] rev 55454
Lifting: support a type variable as a raw type
Thu, 13 Feb 2014 13:16:17 +0100 repaired logic for default provers -- ensures Z3 is kept if installed and configured as noncommercial
blanchet [Thu, 13 Feb 2014 13:16:17 +0100] rev 55453
repaired logic for default provers -- ensures Z3 is kept if installed and configured as noncommercial
Thu, 13 Feb 2014 13:16:17 +0100 avoid changing the state's context -- this results in transfer problems later with SMT, and hence preplay tactic failures
blanchet [Thu, 13 Feb 2014 13:16:17 +0100] rev 55452
avoid changing the state's context -- this results in transfer problems later with SMT, and hence preplay tactic failures
Thu, 13 Feb 2014 13:16:16 +0100 removed hint that is seldom useful in practice
blanchet [Thu, 13 Feb 2014 13:16:16 +0100] rev 55451
removed hint that is seldom useful in practice
Thu, 13 Feb 2014 12:24:28 +0100 reactivate some examples that still appear to work;
wenzelm [Thu, 13 Feb 2014 12:24:28 +0100] rev 55450
reactivate some examples that still appear to work;
Thu, 13 Feb 2014 12:14:47 +0100 removed dead code;
wenzelm [Thu, 13 Feb 2014 12:14:47 +0100] rev 55449
removed dead code;
Thu, 13 Feb 2014 12:09:51 +0100 explicit indication that redefining outer syntax commands is not supposed to happen -- NB: interactive mode requires global change of syntax;
wenzelm [Thu, 13 Feb 2014 12:09:51 +0100] rev 55448
explicit indication that redefining outer syntax commands is not supposed to happen -- NB: interactive mode requires global change of syntax;
Thu, 13 Feb 2014 11:54:14 +0100 do not redefine outer syntax commands;
wenzelm [Thu, 13 Feb 2014 11:54:14 +0100] rev 55447
do not redefine outer syntax commands;
Thu, 13 Feb 2014 11:37:00 +0100 tuned whitespace;
wenzelm [Thu, 13 Feb 2014 11:37:00 +0100] rev 55446
tuned whitespace;
Thu, 13 Feb 2014 11:23:55 +0100 static repair of ML file -- untested (!) by default since 76965c356d2a;
wenzelm [Thu, 13 Feb 2014 11:23:55 +0100] rev 55445
static repair of ML file -- untested (!) by default since 76965c356d2a;
Wed, 12 Feb 2014 17:36:00 +0100 iteration n in the 'default' vs. 'update_new' vs. 'update' saga -- 'update' makes sense now that we honor the canonical order on 'merge' (as opposed to raising 'DUP')
blanchet [Wed, 12 Feb 2014 17:36:00 +0100] rev 55444
iteration n in the 'default' vs. 'update_new' vs. 'update' saga -- 'update' makes sense now that we honor the canonical order on 'merge' (as opposed to raising 'DUP')
Wed, 12 Feb 2014 17:35:59 +0100 don't hide constant forever, since it may appear in some 'primcorec'-generated theorems
blanchet [Wed, 12 Feb 2014 17:35:59 +0100] rev 55443
don't hide constant forever, since it may appear in some 'primcorec'-generated theorems
Wed, 12 Feb 2014 17:35:59 +0100 tuning
blanchet [Wed, 12 Feb 2014 17:35:59 +0100] rev 55442
tuning
Wed, 12 Feb 2014 16:35:58 +0100 HOL-IMP fastness
traytel [Wed, 12 Feb 2014 16:35:58 +0100] rev 55441
HOL-IMP fastness
Wed, 12 Feb 2014 14:32:45 +0100 merged, resolving some conflicts;
wenzelm [Wed, 12 Feb 2014 14:32:45 +0100] rev 55440
merged, resolving some conflicts;
Wed, 12 Feb 2014 13:56:43 +0100 eliminated hard tabs (assuming tab-width=2);
wenzelm [Wed, 12 Feb 2014 13:56:43 +0100] rev 55439
eliminated hard tabs (assuming tab-width=2);
Wed, 12 Feb 2014 13:53:11 +0100 more platform notes;
wenzelm [Wed, 12 Feb 2014 13:53:11 +0100] rev 55438
more platform notes;
Wed, 12 Feb 2014 13:33:05 +0100 tuned whitespace;
wenzelm [Wed, 12 Feb 2014 13:33:05 +0100] rev 55437
tuned whitespace;
Wed, 12 Feb 2014 13:31:18 +0100 removed odd comments -- inferred types are shown by Prover IDE;
wenzelm [Wed, 12 Feb 2014 13:31:18 +0100] rev 55436
removed odd comments -- inferred types are shown by Prover IDE;
Wed, 12 Feb 2014 11:28:17 +0100 maintain blob edits within history, which is important for Snapshot.convert/revert;
wenzelm [Wed, 12 Feb 2014 11:28:17 +0100] rev 55435
maintain blob edits within history, which is important for Snapshot.convert/revert;
Wed, 12 Feb 2014 11:05:48 +0100 more accurate eq_content;
wenzelm [Wed, 12 Feb 2014 11:05:48 +0100] rev 55434
more accurate eq_content;
Wed, 12 Feb 2014 10:50:49 +0100 clarified message_positions: cover alt_id as well;
wenzelm [Wed, 12 Feb 2014 10:50:49 +0100] rev 55433
clarified message_positions: cover alt_id as well; tuned;
Tue, 11 Feb 2014 21:58:31 +0100 maintain multiple command chunks and markup trees: for main chunk and loaded files;
wenzelm [Tue, 11 Feb 2014 21:58:31 +0100] rev 55432
maintain multiple command chunks and markup trees: for main chunk and loaded files; document view for all text areas, including auxiliary files;
Tue, 11 Feb 2014 17:44:29 +0100 common Command.Chunk for command source and auxiliary files (static Symbol.Index without actual String content);
wenzelm [Tue, 11 Feb 2014 17:44:29 +0100] rev 55431
common Command.Chunk for command source and auxiliary files (static Symbol.Index without actual String content); more informative type Blob, to allow markup reports;
Tue, 11 Feb 2014 15:55:05 +0100 tuned signature;
wenzelm [Tue, 11 Feb 2014 15:55:05 +0100] rev 55430
tuned signature;
Tue, 11 Feb 2014 15:05:13 +0100 report (but ignore) markup within auxiliary files;
wenzelm [Tue, 11 Feb 2014 15:05:13 +0100] rev 55429
report (but ignore) markup within auxiliary files;
Wed, 12 Feb 2014 10:59:25 +0100 merged
Andreas Lochbihler [Wed, 12 Feb 2014 10:59:25 +0100] rev 55428
merged
Wed, 12 Feb 2014 09:06:04 +0100 make integer_of_char and char_of_integer work with NBE and code_simp
Andreas Lochbihler [Wed, 12 Feb 2014 09:06:04 +0100] rev 55427
make integer_of_char and char_of_integer work with NBE and code_simp
Wed, 12 Feb 2014 08:56:38 +0100 make lifting setup for String.literal local to prevent transfer from replacing STR ''...'' literals
Andreas Lochbihler [Wed, 12 Feb 2014 08:56:38 +0100] rev 55426
make lifting setup for String.literal local to prevent transfer from replacing STR ''...'' literals
Wed, 12 Feb 2014 10:20:31 +0100 [mq]: news
blanchet [Wed, 12 Feb 2014 10:20:31 +0100] rev 55425
[mq]: news
Wed, 12 Feb 2014 08:37:28 +0100 remove hidden fact about hidden constant from code generator setup
blanchet [Wed, 12 Feb 2014 08:37:28 +0100] rev 55424
remove hidden fact about hidden constant from code generator setup
Wed, 12 Feb 2014 08:37:28 +0100 for extraction -- use the exhaust rule that's registered with 'datatype_realizer.ML'
blanchet [Wed, 12 Feb 2014 08:37:28 +0100] rev 55423
for extraction -- use the exhaust rule that's registered with 'datatype_realizer.ML'
Wed, 12 Feb 2014 08:37:28 +0100 compile
blanchet [Wed, 12 Feb 2014 08:37:28 +0100] rev 55422
compile
Wed, 12 Feb 2014 08:37:28 +0100 updated certificates
blanchet [Wed, 12 Feb 2014 08:37:28 +0100] rev 55421
updated certificates
Wed, 12 Feb 2014 08:37:28 +0100 tuned message
blanchet [Wed, 12 Feb 2014 08:37:28 +0100] rev 55420
tuned message
Wed, 12 Feb 2014 08:37:28 +0100 tabled, v.: postpone consideration of
blanchet [Wed, 12 Feb 2014 08:37:28 +0100] rev 55419
tabled, v.: postpone consideration of
Wed, 12 Feb 2014 08:37:28 +0100 adapted to renaming of 'Projl' and 'Projr'
blanchet [Wed, 12 Feb 2014 08:37:28 +0100] rev 55418
adapted to renaming of 'Projl' and 'Projr'
Wed, 12 Feb 2014 08:37:06 +0100 adapted to 'xxx_{case,rec}' renaming, to new theorem names, and to new variable names in theorems
blanchet [Wed, 12 Feb 2014 08:37:06 +0100] rev 55417
adapted to 'xxx_{case,rec}' renaming, to new theorem names, and to new variable names in theorems * * * more transition of 'xxx_rec' to 'rec_xxx' and same for case * * * compile * * * 'rename_tac's to avoid referring to generated names * * * more robust scripts with 'rename_tac' * * * 'where' -> 'of' * * * 'where' -> 'of' * * * renamed 'xxx_rec' to 'rec_xxx'
Wed, 12 Feb 2014 08:35:57 +0100 adapted theories to 'xxx_case' to 'case_xxx'
blanchet [Wed, 12 Feb 2014 08:35:57 +0100] rev 55416
adapted theories to 'xxx_case' to 'case_xxx' * * * 'char_case' -> 'case_char' and same for 'rec' * * * compile * * * renamed 'xxx_case' to 'case_xxx'
Wed, 12 Feb 2014 08:35:57 +0100 renamed 'nat_{case,rec}' to '{case,rec}_nat'
blanchet [Wed, 12 Feb 2014 08:35:57 +0100] rev 55415
renamed 'nat_{case,rec}' to '{case,rec}_nat'
Wed, 12 Feb 2014 08:35:57 +0100 renamed '{prod,sum,bool,unit}_case' to 'case_...'
blanchet [Wed, 12 Feb 2014 08:35:57 +0100] rev 55414
renamed '{prod,sum,bool,unit}_case' to 'case_...'
Wed, 12 Feb 2014 08:35:56 +0100 adapted theories to '{case,rec}_{list,option}' names
blanchet [Wed, 12 Feb 2014 08:35:56 +0100] rev 55413
adapted theories to '{case,rec}_{list,option}' names
Wed, 12 Feb 2014 08:35:56 +0100 avoid old 'prod.simps' -- better be more specific
blanchet [Wed, 12 Feb 2014 08:35:56 +0100] rev 55412
avoid old 'prod.simps' -- better be more specific
Wed, 12 Feb 2014 08:35:56 +0100 repaired hard-coded constant names
blanchet [Wed, 12 Feb 2014 08:35:56 +0100] rev 55411
repaired hard-coded constant names
Wed, 12 Feb 2014 08:35:56 +0100 killed 'rep_compat' option
blanchet [Wed, 12 Feb 2014 08:35:56 +0100] rev 55410
killed 'rep_compat' option
Wed, 12 Feb 2014 08:35:56 +0100 made 'ctr_sugar' more friendly to the 'datatype_realizer'
blanchet [Wed, 12 Feb 2014 08:35:56 +0100] rev 55409
made 'ctr_sugar' more friendly to the 'datatype_realizer' * * * reverted changes to 'datatype_realizer.ML'
Wed, 12 Feb 2014 08:35:56 +0100 use names like 'rec_mytype' and 'case_mytype' in old datatype package as well, to avoid a mixture
blanchet [Wed, 12 Feb 2014 08:35:56 +0100] rev 55408
use names like 'rec_mytype' and 'case_mytype' in old datatype package as well, to avoid a mixture
Wed, 12 Feb 2014 08:35:56 +0100 use right local theory -- shows up when 'no_discs_sels' is set
blanchet [Wed, 12 Feb 2014 08:35:56 +0100] rev 55407
use right local theory -- shows up when 'no_discs_sels' is set
Wed, 12 Feb 2014 08:35:56 +0100 compatibility names
blanchet [Wed, 12 Feb 2014 08:35:56 +0100] rev 55406
compatibility names
Wed, 12 Feb 2014 08:35:56 +0100 use new selector support to define 'the', 'hd', 'tl'
blanchet [Wed, 12 Feb 2014 08:35:56 +0100] rev 55405
use new selector support to define 'the', 'hd', 'tl'
Wed, 12 Feb 2014 08:35:56 +0100 transformed 'option' and 'list' into new-style datatypes (but register them as old-style as well)
blanchet [Wed, 12 Feb 2014 08:35:56 +0100] rev 55404
transformed 'option' and 'list' into new-style datatypes (but register them as old-style as well) * * * compile * * * tuned imports to prevent merge issues in 'Main'
Wed, 12 Feb 2014 08:35:56 +0100 avoid duplicate 'case' definitions by first looking up 'Ctr_Sugar'
blanchet [Wed, 12 Feb 2014 08:35:56 +0100] rev 55403
avoid duplicate 'case' definitions by first looking up 'Ctr_Sugar'
Wed, 12 Feb 2014 08:35:56 +0100 tuned code
blanchet [Wed, 12 Feb 2014 08:35:56 +0100] rev 55402
tuned code
Wed, 12 Feb 2014 08:35:56 +0100 more 'ctr_sugar' modernization
blanchet [Wed, 12 Feb 2014 08:35:56 +0100] rev 55401
more 'ctr_sugar' modernization
Wed, 12 Feb 2014 08:35:56 +0100 tuning
blanchet [Wed, 12 Feb 2014 08:35:56 +0100] rev 55400
tuning
Wed, 12 Feb 2014 08:35:56 +0100 ported predicate compiler to 'ctr_sugar'
blanchet [Wed, 12 Feb 2014 08:35:56 +0100] rev 55399
ported predicate compiler to 'ctr_sugar' * * * ported predicate compiler to 'ctr_sugar', part 2
Wed, 12 Feb 2014 08:35:56 +0100 updated docs
blanchet [Wed, 12 Feb 2014 08:35:56 +0100] rev 55398
updated docs
Wed, 12 Feb 2014 08:35:56 +0100 generate 'fundec_cong' attribute for new-style (co)datatypes
blanchet [Wed, 12 Feb 2014 08:35:56 +0100] rev 55397
generate 'fundec_cong' attribute for new-style (co)datatypes * * * compile
Wed, 12 Feb 2014 08:35:56 +0100 got rid of dynamic scoping the easy way
blanchet [Wed, 12 Feb 2014 08:35:56 +0100] rev 55396
got rid of dynamic scoping the easy way
Wed, 12 Feb 2014 08:35:56 +0100 removed trivial 'rec' examples for nonrecursive types (I could also have added the 'old.' prefix in front of the constant names)
blanchet [Wed, 12 Feb 2014 08:35:56 +0100] rev 55395
removed trivial 'rec' examples for nonrecursive types (I could also have added the 'old.' prefix in front of the constant names)
Wed, 12 Feb 2014 08:35:56 +0100 more liberal merging of BNFs and constructor sugar
blanchet [Wed, 12 Feb 2014 08:35:56 +0100] rev 55394
more liberal merging of BNFs and constructor sugar * * * make sure that the cache doesn't produce 'DUP's
Wed, 12 Feb 2014 08:35:56 +0100 se 'wrap_free_constructors' to register 'sum' , 'prod', 'unit', 'bool' with their discriminators/selectors
blanchet [Wed, 12 Feb 2014 08:35:56 +0100] rev 55393
se 'wrap_free_constructors' to register 'sum' , 'prod', 'unit', 'bool' with their discriminators/selectors * * * cleaner simp/iff sets
Wed, 12 Feb 2014 08:35:56 +0100 have the same no-update semantics for 'case' as for 'Ctr_Sugar' and BNF data (this might not be the final word on the matter, but using a consistent policy seems like a good idea)
blanchet [Wed, 12 Feb 2014 08:35:56 +0100] rev 55392
have the same no-update semantics for 'case' as for 'Ctr_Sugar' and BNF data (this might not be the final word on the matter, but using a consistent policy seems like a good idea)
Tue, 11 Feb 2014 12:08:44 +0100 Mac OS X Lion (macbroy6) is baseline for portable executables;
wenzelm [Tue, 11 Feb 2014 12:08:44 +0100] rev 55391
Mac OS X Lion (macbroy6) is baseline for portable executables; fringe platforms are unsupported;
Tue, 11 Feb 2014 11:30:33 +0100 "no_memory" option for the simplifier trace to bypass memoization
Lars Hupel <lars.hupel@mytum.de> [Tue, 11 Feb 2014 11:30:33 +0100] rev 55390
"no_memory" option for the simplifier trace to bypass memoization
Tue, 11 Feb 2014 09:29:46 +0100 tuned
nipkow [Tue, 11 Feb 2014 09:29:46 +0100] rev 55389
tuned
Mon, 10 Feb 2014 23:24:44 +0100 merged
wenzelm [Mon, 10 Feb 2014 23:24:44 +0100] rev 55388
merged
Mon, 10 Feb 2014 22:39:04 +0100 seal system channels at end of Pure bootstrap -- Isabelle/Scala provides official interfaces;
wenzelm [Mon, 10 Feb 2014 22:39:04 +0100] rev 55387
seal system channels at end of Pure bootstrap -- Isabelle/Scala provides official interfaces;
(0) -30000 -10000 -3000 -1000 -120 +120 +1000 +3000 +10000 tip