Fri, 14 Feb 2014 15:03:23 +0100 |
blanchet |
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
|
changeset |
files
|
Fri, 14 Feb 2014 14:54:08 +0100 |
traytel |
made N2M more robust w.r.t. identical nested types
|
changeset |
files
|
Fri, 14 Feb 2014 13:45:29 +0100 |
traytel |
register bnfs for (co)datatypes under their proper name (lost in af71b753c459)
|
changeset |
files
|
Fri, 14 Feb 2014 11:10:28 +0100 |
wenzelm |
updated keywords;
|
changeset |
files
|
Fri, 14 Feb 2014 10:33:57 +0100 |
blanchet |
restored old 'remotify' logic -- too many bugs were introduced when refactoring the code
|
changeset |
files
|
Fri, 14 Feb 2014 07:53:46 +0100 |
blanchet |
more (co)datatype docs
|
changeset |
files
|
Fri, 14 Feb 2014 07:53:46 +0100 |
blanchet |
hide 'rel' name -- this one is waiting to be merged with 'list_all2'
|
changeset |
files
|
Fri, 14 Feb 2014 07:53:46 +0100 |
blanchet |
updated docs to reflect the new 'free_constructors' syntax
|
changeset |
files
|
Fri, 14 Feb 2014 07:53:46 +0100 |
blanchet |
more precise spec rules for selectors
|
changeset |
files
|
Fri, 14 Feb 2014 07:53:46 +0100 |
blanchet |
removed needless robustness (no longer needed thanks to new syntax)
|
changeset |
files
|
Fri, 14 Feb 2014 07:53:46 +0100 |
blanchet |
aligned the syntax for 'free_constructors' on the 'datatype_new' and 'codatatype' syntax
|
changeset |
files
|
Fri, 14 Feb 2014 07:53:46 +0100 |
blanchet |
renamed 'wrap_free_constructors' to 'free_constructors' (cf. 'functor', 'bnf', etc.)
|
changeset |
files
|
Fri, 14 Feb 2014 07:53:46 +0100 |
blanchet |
renamed 'enriched_type' to more informative 'functor' (following the renaming of enriched type constructors to bounded natural functors)
|
changeset |
files
|
Fri, 14 Feb 2014 07:53:46 +0100 |
blanchet |
merged 'Option.map' and 'Option.map_option'
|
changeset |
files
|
Fri, 14 Feb 2014 07:53:45 +0100 |
blanchet |
merged 'List.map' and 'List.list.map'
|
changeset |
files
|
Fri, 14 Feb 2014 07:53:45 +0100 |
blanchet |
have 'Ctr_Sugar' register its 'Spec_Rules'
|
changeset |
files
|
Fri, 14 Feb 2014 07:53:45 +0100 |
blanchet |
register 'Spec_Rules' for new-style (co)datatypes
|
changeset |
files
|
Fri, 14 Feb 2014 07:53:45 +0100 |
blanchet |
added 'Spec_Rules' for 'primcorec'
|
changeset |
files
|
Thu, 13 Feb 2014 22:35:38 +0100 |
wenzelm |
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);
|
changeset |
files
|
Thu, 13 Feb 2014 17:11:25 +0100 |
blanchet |
added a bit of documentation for the different commands
|
changeset |
files
|
Thu, 13 Feb 2014 17:11:11 +0100 |
blanchet |
cleaner, complete proof in documentation, contributed by Dmitriy T.
|
changeset |
files
|
Thu, 13 Feb 2014 16:21:43 +0100 |
blanchet |
do the right thing with provers that exist only remotely (e.g. e_sine)
|
changeset |
files
|
Thu, 13 Feb 2014 15:51:54 +0100 |
kuncar |
more precise descripiton
|
changeset |
files
|
Thu, 13 Feb 2014 14:32:05 +0100 |
kuncar |
all_args_conv works also for zero arguments
|
changeset |
files
|
Thu, 13 Feb 2014 14:32:04 +0100 |
kuncar |
don't catch QOUT_THM_INTERNAL from the recursive call of parametrize_relation_conv
|
changeset |
files
|
Wed, 12 Feb 2014 18:32:55 +0100 |
kuncar |
Lifting: support a type variable as a raw type
|
changeset |
files
|
Thu, 13 Feb 2014 13:16:17 +0100 |
blanchet |
repaired logic for default provers -- ensures Z3 is kept if installed and configured as noncommercial
|
changeset |
files
|
Thu, 13 Feb 2014 13:16:17 +0100 |
blanchet |
avoid changing the state's context -- this results in transfer problems later with SMT, and hence preplay tactic failures
|
changeset |
files
|
Thu, 13 Feb 2014 13:16:16 +0100 |
blanchet |
removed hint that is seldom useful in practice
|
changeset |
files
|
Thu, 13 Feb 2014 12:24:28 +0100 |
wenzelm |
reactivate some examples that still appear to work;
|
changeset |
files
|
Thu, 13 Feb 2014 12:14:47 +0100 |
wenzelm |
removed dead code;
|
changeset |
files
|
Thu, 13 Feb 2014 12:09:51 +0100 |
wenzelm |
explicit indication that redefining outer syntax commands is not supposed to happen -- NB: interactive mode requires global change of syntax;
|
changeset |
files
|
Thu, 13 Feb 2014 11:54:14 +0100 |
wenzelm |
do not redefine outer syntax commands;
|
changeset |
files
|
Thu, 13 Feb 2014 11:37:00 +0100 |
wenzelm |
tuned whitespace;
|
changeset |
files
|
Thu, 13 Feb 2014 11:23:55 +0100 |
wenzelm |
static repair of ML file -- untested (!) by default since 76965c356d2a;
|
changeset |
files
|
Wed, 12 Feb 2014 17:36:00 +0100 |
blanchet |
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')
|
changeset |
files
|
Wed, 12 Feb 2014 17:35:59 +0100 |
blanchet |
don't hide constant forever, since it may appear in some 'primcorec'-generated theorems
|
changeset |
files
|
Wed, 12 Feb 2014 17:35:59 +0100 |
blanchet |
tuning
|
changeset |
files
|
Wed, 12 Feb 2014 16:35:58 +0100 |
traytel |
HOL-IMP fastness
|
changeset |
files
|
Wed, 12 Feb 2014 14:32:45 +0100 |
wenzelm |
merged, resolving some conflicts;
|
changeset |
files
|
Wed, 12 Feb 2014 13:56:43 +0100 |
wenzelm |
eliminated hard tabs (assuming tab-width=2);
|
changeset |
files
|
Wed, 12 Feb 2014 13:53:11 +0100 |
wenzelm |
more platform notes;
|
changeset |
files
|
Wed, 12 Feb 2014 13:33:05 +0100 |
wenzelm |
tuned whitespace;
|
changeset |
files
|
Wed, 12 Feb 2014 13:31:18 +0100 |
wenzelm |
removed odd comments -- inferred types are shown by Prover IDE;
|
changeset |
files
|
Wed, 12 Feb 2014 11:28:17 +0100 |
wenzelm |
maintain blob edits within history, which is important for Snapshot.convert/revert;
|
changeset |
files
|
Wed, 12 Feb 2014 11:05:48 +0100 |
wenzelm |
more accurate eq_content;
|
changeset |
files
|
Wed, 12 Feb 2014 10:50:49 +0100 |
wenzelm |
clarified message_positions: cover alt_id as well;
|
changeset |
files
|
Tue, 11 Feb 2014 21:58:31 +0100 |
wenzelm |
maintain multiple command chunks and markup trees: for main chunk and loaded files;
|
changeset |
files
|
Tue, 11 Feb 2014 17:44:29 +0100 |
wenzelm |
common Command.Chunk for command source and auxiliary files (static Symbol.Index without actual String content);
|
changeset |
files
|
Tue, 11 Feb 2014 15:55:05 +0100 |
wenzelm |
tuned signature;
|
changeset |
files
|
Tue, 11 Feb 2014 15:05:13 +0100 |
wenzelm |
report (but ignore) markup within auxiliary files;
|
changeset |
files
|
Wed, 12 Feb 2014 10:59:25 +0100 |
Andreas Lochbihler |
merged
|
changeset |
files
|
Wed, 12 Feb 2014 09:06:04 +0100 |
Andreas Lochbihler |
make integer_of_char and char_of_integer work with NBE and code_simp
|
changeset |
files
|
Wed, 12 Feb 2014 08:56:38 +0100 |
Andreas Lochbihler |
make lifting setup for String.literal local to prevent transfer from replacing STR ''...'' literals
|
changeset |
files
|
Wed, 12 Feb 2014 10:20:31 +0100 |
blanchet |
[mq]: news
|
changeset |
files
|
Wed, 12 Feb 2014 08:37:28 +0100 |
blanchet |
remove hidden fact about hidden constant from code generator setup
|
changeset |
files
|
Wed, 12 Feb 2014 08:37:28 +0100 |
blanchet |
for extraction -- use the exhaust rule that's registered with 'datatype_realizer.ML'
|
changeset |
files
|
Wed, 12 Feb 2014 08:37:28 +0100 |
blanchet |
compile
|
changeset |
files
|
Wed, 12 Feb 2014 08:37:28 +0100 |
blanchet |
updated certificates
|
changeset |
files
|
Wed, 12 Feb 2014 08:37:28 +0100 |
blanchet |
tuned message
|
changeset |
files
|
Wed, 12 Feb 2014 08:37:28 +0100 |
blanchet |
tabled, v.: postpone consideration of
|
changeset |
files
|
Wed, 12 Feb 2014 08:37:28 +0100 |
blanchet |
adapted to renaming of 'Projl' and 'Projr'
|
changeset |
files
|
Wed, 12 Feb 2014 08:37:06 +0100 |
blanchet |
adapted to 'xxx_{case,rec}' renaming, to new theorem names, and to new variable names in theorems
|
changeset |
files
|
Wed, 12 Feb 2014 08:35:57 +0100 |
blanchet |
adapted theories to 'xxx_case' to 'case_xxx'
|
changeset |
files
|
Wed, 12 Feb 2014 08:35:57 +0100 |
blanchet |
renamed 'nat_{case,rec}' to '{case,rec}_nat'
|
changeset |
files
|
Wed, 12 Feb 2014 08:35:57 +0100 |
blanchet |
renamed '{prod,sum,bool,unit}_case' to 'case_...'
|
changeset |
files
|
Wed, 12 Feb 2014 08:35:56 +0100 |
blanchet |
adapted theories to '{case,rec}_{list,option}' names
|
changeset |
files
|
Wed, 12 Feb 2014 08:35:56 +0100 |
blanchet |
avoid old 'prod.simps' -- better be more specific
|
changeset |
files
|
Wed, 12 Feb 2014 08:35:56 +0100 |
blanchet |
repaired hard-coded constant names
|
changeset |
files
|
Wed, 12 Feb 2014 08:35:56 +0100 |
blanchet |
killed 'rep_compat' option
|
changeset |
files
|
Wed, 12 Feb 2014 08:35:56 +0100 |
blanchet |
made 'ctr_sugar' more friendly to the 'datatype_realizer'
|
changeset |
files
|
Wed, 12 Feb 2014 08:35:56 +0100 |
blanchet |
use names like 'rec_mytype' and 'case_mytype' in old datatype package as well, to avoid a mixture
|
changeset |
files
|
Wed, 12 Feb 2014 08:35:56 +0100 |
blanchet |
use right local theory -- shows up when 'no_discs_sels' is set
|
changeset |
files
|
Wed, 12 Feb 2014 08:35:56 +0100 |
blanchet |
compatibility names
|
changeset |
files
|
Wed, 12 Feb 2014 08:35:56 +0100 |
blanchet |
use new selector support to define 'the', 'hd', 'tl'
|
changeset |
files
|
Wed, 12 Feb 2014 08:35:56 +0100 |
blanchet |
transformed 'option' and 'list' into new-style datatypes (but register them as old-style as well)
|
changeset |
files
|
Wed, 12 Feb 2014 08:35:56 +0100 |
blanchet |
avoid duplicate 'case' definitions by first looking up 'Ctr_Sugar'
|
changeset |
files
|
Wed, 12 Feb 2014 08:35:56 +0100 |
blanchet |
tuned code
|
changeset |
files
|
Wed, 12 Feb 2014 08:35:56 +0100 |
blanchet |
more 'ctr_sugar' modernization
|
changeset |
files
|
Wed, 12 Feb 2014 08:35:56 +0100 |
blanchet |
tuning
|
changeset |
files
|
Wed, 12 Feb 2014 08:35:56 +0100 |
blanchet |
ported predicate compiler to 'ctr_sugar'
|
changeset |
files
|
Wed, 12 Feb 2014 08:35:56 +0100 |
blanchet |
updated docs
|
changeset |
files
|
Wed, 12 Feb 2014 08:35:56 +0100 |
blanchet |
generate 'fundec_cong' attribute for new-style (co)datatypes
|
changeset |
files
|
Wed, 12 Feb 2014 08:35:56 +0100 |
blanchet |
got rid of dynamic scoping the easy way
|
changeset |
files
|
Wed, 12 Feb 2014 08:35:56 +0100 |
blanchet |
removed trivial 'rec' examples for nonrecursive types (I could also have added the 'old.' prefix in front of the constant names)
|
changeset |
files
|
Wed, 12 Feb 2014 08:35:56 +0100 |
blanchet |
more liberal merging of BNFs and constructor sugar
|
changeset |
files
|
Wed, 12 Feb 2014 08:35:56 +0100 |
blanchet |
se 'wrap_free_constructors' to register 'sum' , 'prod', 'unit', 'bool' with their discriminators/selectors
|
changeset |
files
|
Wed, 12 Feb 2014 08:35:56 +0100 |
blanchet |
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)
|
changeset |
files
|
Tue, 11 Feb 2014 12:08:44 +0100 |
wenzelm |
Mac OS X Lion (macbroy6) is baseline for portable executables;
|
changeset |
files
|
Tue, 11 Feb 2014 11:30:33 +0100 |
Lars Hupel |
"no_memory" option for the simplifier trace to bypass memoization
|
changeset |
files
|
Tue, 11 Feb 2014 09:29:46 +0100 |
nipkow |
tuned
|
changeset |
files
|
Mon, 10 Feb 2014 23:24:44 +0100 |
wenzelm |
merged
|
changeset |
files
|
Mon, 10 Feb 2014 22:39:04 +0100 |
wenzelm |
seal system channels at end of Pure bootstrap -- Isabelle/Scala provides official interfaces;
|
changeset |
files
|
Mon, 10 Feb 2014 22:22:06 +0100 |
wenzelm |
make triple-sure that the future scheduler is properly shutdown (see also 702278df3b57);
|
changeset |
files
|
Mon, 10 Feb 2014 22:08:18 +0100 |
wenzelm |
discontinued axiomatic 'classes', 'classrel', 'arities';
|
changeset |
files
|
Mon, 10 Feb 2014 22:07:50 +0100 |
wenzelm |
updated keywords;
|
changeset |
files
|
Mon, 10 Feb 2014 21:03:28 +0100 |
wenzelm |
more explicit axiomatization;
|
changeset |
files
|
Mon, 10 Feb 2014 21:00:56 +0100 |
wenzelm |
prefer vacuous definitional type classes over axiomatic ones;
|
changeset |
files
|
Mon, 10 Feb 2014 17:23:13 +0100 |
wenzelm |
more explicit axiomatization;
|
changeset |
files
|
Mon, 10 Feb 2014 17:20:11 +0100 |
wenzelm |
prefer vacuous definitional type classes over axiomatic ones;
|
changeset |
files
|
Mon, 10 Feb 2014 14:33:47 +0100 |
wenzelm |
comments;
|
changeset |
files
|
Mon, 10 Feb 2014 13:47:31 +0100 |
wenzelm |
removed rotten code;
|
changeset |
files
|
Mon, 10 Feb 2014 13:04:08 +0100 |
wenzelm |
more elementary put_simpset: exchange the simplifier configuration outright, which is particularly relevant concerning cumulative depth, e.g. for Product_Type.split_beta in the subsequent example:
|
changeset |
files
|
Mon, 10 Feb 2014 21:51:15 +0100 |
nipkow |
merged
|
changeset |
files
|
Mon, 10 Feb 2014 21:50:50 +0100 |
nipkow |
improved lin.arith. for terms involving division
|
changeset |
files
|
Sun, 09 Feb 2014 21:37:27 +0100 |
haftmann |
restoring ancient string_classes option
|
changeset |
files
|
Sun, 09 Feb 2014 21:37:27 +0100 |
haftmann |
method names in instance declarations are always unqualified
|
changeset |
files
|
Sun, 09 Feb 2014 21:37:27 +0100 |
haftmann |
dropped legacy finally
|
changeset |
files
|
Sun, 09 Feb 2014 19:10:12 +0000 |
paulson |
tidied messy proofs
|
changeset |
files
|
Sun, 09 Feb 2014 17:47:23 +0100 |
wenzelm |
minimal document;
|
changeset |
files
|
Sun, 09 Feb 2014 17:41:17 +0100 |
wenzelm |
removed junk;
|
changeset |
files
|
Sun, 09 Feb 2014 17:21:03 +0100 |
wenzelm |
merged
|
changeset |
files
|
Sun, 09 Feb 2014 17:19:22 +0100 |
wenzelm |
check scalable fonts;
|
changeset |
files
|
Sun, 09 Feb 2014 16:31:24 +0100 |
wenzelm |
do *not* enforce scalable fonts for T1 encoding, instead rely on cm-super fonts, which also provide underscore for non-tt font;
|
changeset |
files
|
Sun, 09 Feb 2014 16:17:01 +0100 |
wenzelm |
yet another attempt at actual underscore;
|
changeset |
files
|
Sun, 09 Feb 2014 15:26:33 +0100 |
haftmann |
build up preprocessing context only once
|
changeset |
files
|
Sun, 09 Feb 2014 15:26:33 +0100 |
haftmann |
tuned
|
changeset |
files
|
Sun, 09 Feb 2014 13:07:23 +0100 |
nipkow |
disabled counterexample output for now; confusing because often incorrect
|
changeset |
files
|
Sat, 08 Feb 2014 20:34:10 +0100 |
nipkow |
more indexing
|
changeset |
files
|
Fri, 07 Feb 2014 22:37:54 +0100 |
nipkow |
merged
|
changeset |
files
|