merged
authornipkow
Mon, 16 Apr 2012 19:01:57 +0200
changeset 47495 573ca05db948
parent 47494 8c8f27864ed1 (diff)
parent 47493 2feb0aab030f (current diff)
child 47496 a43f207f216f
merged
NEWS
doc-src/IsarOverview/IsaMakefile
doc-src/IsarOverview/Isar/Induction.thy
doc-src/IsarOverview/Isar/Logic.thy
doc-src/IsarOverview/Isar/ROOT.ML
doc-src/IsarOverview/Isar/document/Induction.tex
doc-src/IsarOverview/Isar/document/Logic.tex
doc-src/IsarOverview/Isar/document/Makefile
doc-src/IsarOverview/Isar/document/intro.tex
doc-src/IsarOverview/Isar/document/llncs.cls
doc-src/IsarOverview/Isar/document/root.bib
doc-src/IsarOverview/Isar/document/root.tex
doc-src/IsarOverview/Isar/makeDemo
doc-src/IsarOverview/Makefile
src/HOL/Mirabelle/Tools/mirabelle.ML
src/HOL/Mirabelle/Tools/mirabelle_arith.ML
src/HOL/Mirabelle/Tools/mirabelle_metis.ML
src/HOL/Mirabelle/Tools/mirabelle_quickcheck.ML
src/HOL/Mirabelle/Tools/mirabelle_refute.ML
src/HOL/Mirabelle/Tools/mirabelle_sledgehammer.ML
src/HOL/Mirabelle/Tools/mirabelle_sledgehammer_filter.ML
src/HOL/ex/Set_Algebras.thy
--- a/NEWS	Mon Apr 16 17:26:32 2012 +0200
+++ b/NEWS	Mon Apr 16 19:01:57 2012 +0200
@@ -129,10 +129,39 @@
 
 *** HOL ***
 
-* New tutorial Programming and Proving in Isabelle/HOL ("prog-prove").
+
+* New tutorial "Programming and Proving in Isabelle/HOL" ("prog-prove").
+It completely supercedes "A Tutorial Introduction to Structured Isar Proofs",
+which has been removed. It supercedes "Isabelle/HOL, A Proof Assistant
+for Higher-Order Logic" as the recommended beginners tutorial
+but does not cover all of the material of that old tutorial.
 
 * Discontinued old Tutorial on Isar ("isar-overview");
 
+* The representation of numerals has changed. We now have a datatype
+"num" representing strictly positive binary numerals, along with
+functions "numeral :: num => 'a" and "neg_numeral :: num => 'a" to
+represent positive and negated numeric literals, respectively. (See
+definitions in Num.thy.) Potential INCOMPATIBILITY; some user theories
+may require adaptations:
+
+  - Theorems with number_ring or number_semiring constraints: These
+    classes are gone; use comm_ring_1 or comm_semiring_1 instead.
+
+  - Theories defining numeric types: Remove number, number_semiring,
+    and number_ring instances. Defer all theorems about numerals until
+    after classes one and semigroup_add have been instantiated.
+
+  - Numeral-only simp rules: Replace each rule having a "number_of v"
+    pattern with two copies, one for numeral and one for neg_numeral.
+
+  - Theorems about subclasses of semiring_1 or ring_1: These classes
+    automatically support numerals now, so more simp rules and
+    simprocs may now apply within the proof.
+
+  - Definitions and theorems using old constructors Pls/Min/Bit0/Bit1:
+    Redefine using other integer operations.
+
 * Type 'a set is now a proper type constructor (just as before
 Isabelle2008).  Definitions mem_def and Collect_def have disappeared.
 Non-trivial INCOMPATIBILITY.  For developments keeping predicates and