NEWS
changeset 17533 f22f2ffd78ba
parent 17519 9c10585a238c
child 17535 cd0a4847d0b8
equal deleted inserted replaced
17532:ab75f2b0cec6 17533:f22f2ffd78ba
   357 patterns (these are not perfect but work quite well):
   357 patterns (these are not perfect but work quite well):
   358 
   358 
   359   {)\([^\.]*\)\.\.  ->  {\1<\.\.}
   359   {)\([^\.]*\)\.\.  ->  {\1<\.\.}
   360   \.\.\([^(}]*\)(}  ->  \.\.<\1}
   360   \.\.\([^(}]*\)(}  ->  \.\.<\1}
   361 
   361 
   362 * Method comm_ring for proving equalities in commutative rings.
   362 * Theory Commutative_Ring (in Library): method comm_ring for proving
       
   363 equalities in commutative rings; method 'algebra' provides a generic
       
   364 interface.
   363 
   365 
   364 * Theory Finite_Set: changed the syntax for 'setsum', summation over
   366 * Theory Finite_Set: changed the syntax for 'setsum', summation over
   365 finite sets: "setsum (%x. e) A", which used to be "\<Sum>x:A. e", is
   367 finite sets: "setsum (%x. e) A", which used to be "\<Sum>x:A. e", is
   366 now either "SUM x:A. e" or "\<Sum>x \<in> A. e". The bound variable can
   368 now either "SUM x:A. e" or "\<Sum>x \<in> A. e". The bound variable can
   367 be a tuple pattern.
   369 be a tuple pattern.
   640 standard variables must have explicit universal quantifiers.
   642 standard variables must have explicit universal quantifiers.
   641 
   643 
   642 
   644 
   643 *** HOLCF ***
   645 *** HOLCF ***
   644 
   646 
   645 * HOLCF: discontinued special version of 'constdefs' (which used to
   647 * Discontinued special version of 'constdefs' (which used to support
   646 support continuous functions) in favor of the general Pure one with
   648 continuous functions) in favor of the general Pure one with full
   647 full type-inference.
   649 type-inference.
   648 
   650 
   649 * HOLCF: new simplification procedure for solving continuity conditions;
   651 * New simplification procedure for solving continuity conditions; it
   650 it is much faster on terms with many nested lambda abstractions (cubic
   652 is much faster on terms with many nested lambda abstractions (cubic
   651 instead of exponential time).
   653 instead of exponential time).
   652 
   654 
   653 * HOLCF: new syntax for domain package: selector names are now optional.
   655 * New syntax for domain package: selector names are now optional.
   654 Parentheses should be omitted unless argument is lazy, for example:
   656 Parentheses should be omitted unless argument is lazy, for example:
   655 
   657 
   656   domain 'a stream = cons "'a" (lazy "'a stream")
   658   domain 'a stream = cons "'a" (lazy "'a stream")
   657 
   659 
   658 * HOLCF: new command "fixrec" for defining recursive functions with pattern
   660 * New command 'fixrec' for defining recursive functions with pattern
   659 matching; defining multiple functions with mutual recursion is also supported.
   661 matching; defining multiple functions with mutual recursion is also
   660 Patterns may include the constants cpair, spair, up, sinl, sinr, or any data
   662 supported.  Patterns may include the constants cpair, spair, up, sinl,
   661 constructor defined by the domain package. The given equations are proven as
   663 sinr, or any data constructor defined by the domain package. The given
   662 rewrite rules. See HOLCF/ex/Fixrec_ex.thy for syntax and examples.
   664 equations are proven as rewrite rules. See HOLCF/ex/Fixrec_ex.thy for
   663 
   665 syntax and examples.
   664 * HOLCF: new commands "cpodef" and "pcpodef" for defining predicate subtypes
   666 
   665 of cpo and pcpo types. Syntax is exactly like the "typedef" command, but the
   667 * New commands 'cpodef' and 'pcpodef' for defining predicate subtypes
   666 proof obligation additionally includes an admissibility requirement. The
   668 of cpo and pcpo types. Syntax is exactly like the 'typedef' command,
   667 packages generate instances of class cpo or pcpo, with continuity and
   669 but the proof obligation additionally includes an admissibility
   668 strictness theorems for Rep and Abs.
   670 requirement. The packages generate instances of class cpo or pcpo,
       
   671 with continuity and strictness theorems for Rep and Abs.
   669 
   672 
   670 
   673 
   671 *** ZF ***
   674 *** ZF ***
   672 
   675 
   673 * ZF/ex: theories Group and Ring provide examples in abstract algebra,
   676 * ZF/ex: theories Group and Ring provide examples in abstract algebra,