NEWS
changeset 22971 a6812b6a36a5
parent 22965 b81bbe298406
child 22972 3e96b98d37c6
--- a/NEWS	Mon May 14 18:48:24 2007 +0200
+++ b/NEWS	Mon May 14 19:14:50 2007 +0200
@@ -868,6 +868,12 @@
 feature is used only for decision, for compatibility with arith. This
 means a goal is either solved or left unchanged, no simplification.
 
+* Hyperreal: Functions root and sqrt are now defined on negative real
+inputs so that root n (- x) = - root n x and sqrt (- x) = - sqrt x.
+Nonnegativity side conditions have been removed from many lemmas, so
+that more subgoals may now be solved by simplification; potential
+INCOMPATIBILITY.
+
 * Real: New axiomatic classes formalize real normed vector spaces and
 algebras, using new overloaded constants scaleR :: real => 'a => 'a
 and norm :: 'a => real.