2014-02-15 wenzelm isabelle-ml mode with separate token marker;
2014-02-15 wenzelm partial scans via ML_Lex.tokenize_context;
2014-02-14 wenzelm proper signature;
2014-02-14 wenzelm lexical syntax for SML (in Scala);
2014-02-14 wenzelm tuned;
2014-02-14 wenzelm removed dead code;
2014-02-14 wenzelm tuned signature (in accordance to ML version);
2014-02-14 wenzelm tuned proofs;
2014-02-14 wenzelm tuned signature -- separate Lexicon from Parsers (in accordance to ML version);
2014-02-14 wenzelm prefer latest ProofGeneral-4.2-1 by default;
2014-02-14 wenzelm updated thy_info.dependencies;
2014-02-14 wenzelm tuned message;
2014-02-14 wenzelm more integrity checks of theory names vs. full node names;
2014-02-14 kuncar abstract type must be a type constructor; check it
2014-02-14 blanchet generate proper 'DtRec' indices in 'datatype_new_compat' for the case where some types are duplicated
2014-02-14 blanchet better handling of recursion through functions
2014-02-14 blanchet added examples/tests
2014-02-14 blanchet tuned code to allow mutualized corecursion through different functions with the same target type
2014-02-14 blanchet removed assumption in 'primrec_new' that a given constructor can only occur once
2014-02-14 blanchet generate unique names
2014-02-14 blanchet allow different functions to recurse on the same type, like in the old package
2014-02-14 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
2014-02-14 traytel made N2M more robust w.r.t. identical nested types
2014-02-14 traytel register bnfs for (co)datatypes under their proper name (lost in af71b753c459)
2014-02-14 wenzelm updated keywords;
2014-02-14 blanchet restored old 'remotify' logic -- too many bugs were introduced when refactoring the code
2014-02-14 blanchet more (co)datatype docs
2014-02-14 blanchet hide 'rel' name -- this one is waiting to be merged with 'list_all2'
2014-02-14 blanchet updated docs to reflect the new 'free_constructors' syntax
2014-02-14 blanchet more precise spec rules for selectors
2014-02-14 blanchet removed needless robustness (no longer needed thanks to new syntax)
2014-02-14 blanchet aligned the syntax for 'free_constructors' on the 'datatype_new' and 'codatatype' syntax
2014-02-14 blanchet renamed 'wrap_free_constructors' to 'free_constructors' (cf. 'functor', 'bnf', etc.)
2014-02-14 blanchet renamed 'enriched_type' to more informative 'functor' (following the renaming of enriched type constructors to bounded natural functors)
2014-02-14 blanchet merged 'Option.map' and 'Option.map_option'
2014-02-14 blanchet merged 'List.map' and 'List.list.map'
2014-02-14 blanchet have 'Ctr_Sugar' register its 'Spec_Rules'
2014-02-14 blanchet register 'Spec_Rules' for new-style (co)datatypes
2014-02-14 blanchet added 'Spec_Rules' for 'primcorec'
2014-02-13 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);
2014-02-13 blanchet added a bit of documentation for the different commands
2014-02-13 blanchet cleaner, complete proof in documentation, contributed by Dmitriy T.
2014-02-13 blanchet do the right thing with provers that exist only remotely (e.g. e_sine)
2014-02-13 kuncar more precise descripiton
2014-02-13 kuncar all_args_conv works also for zero arguments
2014-02-13 kuncar don't catch QOUT_THM_INTERNAL from the recursive call of parametrize_relation_conv
2014-02-12 kuncar Lifting: support a type variable as a raw type
2014-02-13 blanchet repaired logic for default provers -- ensures Z3 is kept if installed and configured as noncommercial
2014-02-13 blanchet avoid changing the state's context -- this results in transfer problems later with SMT, and hence preplay tactic failures
2014-02-13 blanchet removed hint that is seldom useful in practice
2014-02-13 wenzelm reactivate some examples that still appear to work;
2014-02-13 wenzelm removed dead code;
2014-02-13 wenzelm explicit indication that redefining outer syntax commands is not supposed to happen -- NB: interactive mode requires global change of syntax;
2014-02-13 wenzelm do not redefine outer syntax commands;
2014-02-13 wenzelm tuned whitespace;
2014-02-13 wenzelm static repair of ML file -- untested (!) by default since 76965c356d2a;
2014-02-12 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')
2014-02-12 blanchet don't hide constant forever, since it may appear in some 'primcorec'-generated theorems
2014-02-12 blanchet tuning
2014-02-12 traytel HOL-IMP fastness
(0) -30000 -10000 -3000 -1000 -300 -100 -60 +60 +100 +300 +1000 +3000 +10000 tip