# HG changeset patch # User paulson # Date 1402667399 -3600 # Node ID 6515cf25de13e77cb54db8aa9565a7a5abcd957c # Parent 19b7ace1c5da23081c70e1786c66d1b892de384f NEWS diff -r 19b7ace1c5da -r 6515cf25de13 NEWS --- a/NEWS Fri Jun 13 14:08:20 2014 +0200 +++ b/NEWS Fri Jun 13 14:49:59 2014 +0100 @@ -479,7 +479,7 @@ For min_ac or max_ac, prefer more general collection ac_simps. -INCOMPATBILITY. +INCOMPATBILITY. * Word library: bit representations prefer type bool over type bit. INCOMPATIBILITY. @@ -675,6 +675,8 @@ * HOL-Multivariate_Analysis: - type class ordered_real_vector for ordered vector spaces + - new theory Complex_Basic_Analysis defining complex derivatives, + holomorphic functions, etc., ported from HOL Light's canal.ml. - changed order of ordered_euclidean_space to be compatible with pointwise ordering on products. Therefore instance of conditionally_complete_lattice and ordered_real_vector. @@ -6308,7 +6310,7 @@ type and generates all solutions by Prolog-style backward 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)" @@ -7080,7 +7082,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. @@ -7119,7 +7121,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 @@ -7485,7 +7487,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 @@ -7569,7 +7571,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 @@ -8465,19 +8467,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.