tuned;
authorwenzelm
Fri, 24 Jul 2020 16:45:20 +0200
changeset 72070 b17be02a0a11
parent 72069 ebf3ba74bc4c
child 72071 d3cad9ecd0cc
tuned;
NEWS
--- a/NEWS	Fri Jul 24 15:20:35 2020 +0200
+++ b/NEWS	Fri Jul 24 16:45:20 2020 +0200
@@ -37,6 +37,12 @@
 * Session HOL-Examples contains notable examples for Isabelle/HOL
 (former entries of HOL-Isar_Examples, HOL-ex etc.).
 
+* Simproc "defined_all" and rewrite rule "subst_all" perform more
+aggressive substitution with variables from assumptions.
+INCOMPATIBILITY, consider repairing proofs locally like this:
+
+  supply subst_all [simp del] [[simproc del: defined_all]]
+
 * Simproc "datatype_no_proper_subterm" rewrites equalities "lhs = rhs"
 on datatypes to "False" if either side is a proper subexpression of the
 other (for any datatype with a reasonable size function).
@@ -85,26 +91,17 @@
 into theories Misc_lsb, Misc_msb and Misc_set_bit respectively.
 INCOMPATIBILITY.
 
-* Session HOL-TPTP: The "tptp_isabelle" and "tptp_sledgehammer"
-commands are in working order again, as opposed to outputting
-"GaveUp" on nearly all problems.
-
-* Simproc defined_all and rewrite rule subst_all perform
-more aggressive substitution with variables from assumptions.
-INCOMPATIBILITY, use something like
-"supply subst_all [simp del] [[simproc del: defined_all]]"
-to leave fragile proofs unaffected.
+* Session HOL-TPTP: The "tptp_isabelle" and "tptp_sledgehammer" commands
+are in working order again, as opposed to outputting "GaveUp" on nearly
+all problems.
 
 
 *** FOL ***
 
 * Added the "at most 1" quantifier, Uniq, as in HOL.
 
-* Simproc defined_all and rewrite rule subst_all perform
-more aggressive substitution with variables from assumptions.
-INCOMPATIBILITY, use something like
-"supply subst_all [simp del] [[simproc del: defined_all]]"
-to leave fragile proofs unaffected.
+* Simproc "defined_all" and rewrite rule "subst_all" have been changed
+as in HOL.
 
 
 *** ML ***