# HG changeset patch # User blanchet # Date 1346167045 -7200 # Node ID ae12b92c145a84f78670ea3fdd6230e03330ff09 # Parent 2d17c305f4bcc4c057b96bc1ed8705719e6fbbfa updated NEWS and CONTRIBUTORS diff -r 2d17c305f4bc -r ae12b92c145a CONTRIBUTORS --- a/CONTRIBUTORS Tue Aug 28 17:17:03 2012 +0200 +++ b/CONTRIBUTORS Tue Aug 28 17:17:25 2012 +0200 @@ -6,6 +6,12 @@ Contributions to this Isabelle version -------------------------------------- +* August 2012: Dmitriy Traytel, Andrei Popescu, Jasmin Blanchette, TUM + New (co)datatype package. + +* August 2012: Andrei Popescu and Dmitriy Traytel, TUM + Theories of ordinals and cardinals. + * July 2012: Makarius Wenzel, Université Paris-Sud / LRI Advanced support for Isabelle sessions and build management, notably "isabelle build". @@ -161,7 +167,7 @@ * November 2009: Lukas Bulwahn, TUM Predicate Compiler: a compiler for inductive predicates to equational specifications. - + * November 2009: Sascha Boehme, TUM and Burkhart Wolff, LRI Paris HOL-Boogie: an interactive prover back-end for Boogie and VCC. diff -r 2d17c305f4bc -r ae12b92c145a NEWS --- a/NEWS Tue Aug 28 17:17:03 2012 +0200 +++ b/NEWS Tue Aug 28 17:17:25 2012 +0200 @@ -41,6 +41,12 @@ *** HOL *** +* HOL/Codatatype: New (co)datatype package with support for mixed, +nested recursion and interesting non-free datatypes. + +* HOL/Ordinals_and_Cardinals: Theories of ordinals and cardinals +(supersedes the AFP entry of the same name). + * Library/Debug.thy and Library/Parallel.thy: debugging and parallel execution for code generated towards Isabelle/ML. @@ -51,7 +57,7 @@ - added an optimisation for equality premises. It is switched on by default, and can be switched off by setting - the configuration quickcheck_optimise_equality to false. + the configuration quickcheck_optimise_equality to false. * The SMT solver Z3 has now by default a restricted set of directly supported features. For the full set of features (div/mod, nonlinear @@ -4557,7 +4563,7 @@ type and generates all solutions by prolog-style backwards proof using the declared rules. -This setup also deals with rules like +This setup also deals with rules like "is_measure f ==> is_measure (list_size f)" @@ -5329,7 +5335,7 @@ rewrites now. That is, trace_simp_depth_limit is set to 1 by default. Thus there is less danger of being flooded by the trace. The trace indicates where parts have been suppressed. - + * Provers/classical: removed obsolete classical version of elim_format attribute; classical elim/dest rules are now treated uniformly when manipulating the claset. @@ -5368,7 +5374,7 @@ Examples are in the directory MetisExamples. WARNING: the Isabelle/HOL-Metis integration does not yet work properly with multi-threading. - + * Command 'sledgehammer' invokes external automatic theorem provers as background processes. It generates calls to the "metis" method if successful. These can be pasted into the proof. Users do not have to @@ -5734,7 +5740,7 @@ users are encouraged to use the new package. * Method "lexicographic_order" automatically synthesizes termination -relations as lexicographic combinations of size measures. +relations as lexicographic combinations of size measures. * Case-expressions allow arbitrary constructor-patterns (including "_") and take their order into account, like in functional @@ -5818,7 +5824,7 @@ (K x) r The K-combinator that is internally used is called K_record. INCOMPATIBILITY: Usage of the plain update functions has to be adapted. - + * Class "semiring_0" now contains annihilation axioms x * 0 = 0 and 0 * x = 0, which are required for a semiring. Richer structures do not inherit from semiring_0 anymore, because this property is a theorem @@ -6714,19 +6720,19 @@ mult_neg_le now named mult_nonpos_nonpos * The following lemmas in Ring_and_Field have been added to the simplifier: - + zero_le_square - not_square_less_zero + not_square_less_zero The following lemmas have been deleted from Real/RealPow: - + realpow_zero_zero realpow_two realpow_less zero_le_power realpow_two_le abs_realpow_two - realpow_two_abs + realpow_two_abs * Theory Parity: added rules for simplifying exponents.