--- a/ANNOUNCE Sat Apr 14 12:36:11 2012 +0200
+++ b/ANNOUNCE Sat Apr 14 12:46:45 2012 +0200
@@ -1,29 +1,15 @@
-Subject: Announcing Isabelle2011-1
+Subject: Announcing Isabelle2012
To: isabelle-users@cl.cam.ac.uk
-Isabelle2011-1 is now available.
+Isabelle2012 is now available.
-This version significantly improves upon Isabelle2011, see the NEWS
+This version significantly improves upon Isabelle2011-1, see the NEWS
file in the distribution for more details. Some notable changes are:
-* Significantly improved Isabelle/jEdit Prover IDE (PIDE).
-
-* Improved system integration with Isabelle/Scala: YXML data encoding.
-
-* Improved parallel performance and scalability.
-
-* Improved document preparation: embedded rail-road diagrams.
-
-* HOL tool enhancements: Quickcheck, Nitpick, Sledgehammer, SMT/Z3
- integration.
-
-* Numerous HOL library improvements: main HOL, HOLCF, HOL-Library,
- Multivariate_Analysis, Probability.
-
-* Updated and extended Isabelle/Isar reference manual.
+* FIXME
-You may get Isabelle2011-1 from the following mirror sites:
+You may get Isabelle2012 from the following mirror sites:
Cambridge (UK) http://www.cl.cam.ac.uk/research/hvg/Isabelle/
Munich (Germany) http://isabelle.in.tum.de/
--- a/CONTRIBUTORS Sat Apr 14 12:36:11 2012 +0200
+++ b/CONTRIBUTORS Sat Apr 14 12:46:45 2012 +0200
@@ -3,21 +3,25 @@
who is listed as an author in one of the source files of this Isabelle
distribution.
-Contributions to this Isabelle version
---------------------------------------
+Contributions to Isabelle2012
+-----------------------------
-* March 2012: Christian Sternagel, Japan Advanced Institute of Science and Technology
+* March 2012: Christian Sternagel, Japan Advanced Institute of Science
+ and Technology
Consolidated theory of relation composition.
* March 2012: Nik Sultana, University of Cambridge
HOL/TPTP parser and import facilities.
+* March 2012: Cezary Kaliszyk, University of Innsbruck and
+ Alexander Krauss, QAware GmbH
+ Faster and more scalable Import mechanism for HOL Light proofs.
+
* January 2012: Florian Haftmann, TUM, et. al.
(Re-)Introduction of the "set" type constructor.
-* March 2012: Cezary Kaliszyk, University of Innsbruck and
- Alexander Krauss, QAware GmbH
- Faster and more scalable Import mechanism for HOL Light proofs.
+* 2011/2012: Makarius Wenzel, Université Paris-Sud / LRI
+ Improvements of Isabelle/Scala layer and Isabelle/jEdit Prover IDE.
Contributions to Isabelle2011-1
--- a/COPYRIGHT Sat Apr 14 12:36:11 2012 +0200
+++ b/COPYRIGHT Sat Apr 14 12:46:45 2012 +0200
@@ -1,6 +1,6 @@
ISABELLE COPYRIGHT NOTICE, LICENCE AND DISCLAIMER.
-Copyright (c) 2011,
+Copyright (c) 2012,
University of Cambridge,
Technische Universitaet Muenchen,
and contributors.
--- a/NEWS Sat Apr 14 12:36:11 2012 +0200
+++ b/NEWS Sat Apr 14 12:46:45 2012 +0200
@@ -1,8 +1,8 @@
Isabelle NEWS -- history user-relevant changes
==============================================
-New in this Isabelle version
-----------------------------
+New in Isabelle2012 (May 2012)
+------------------------------
*** General ***
@@ -95,7 +95,7 @@
lemma "P (x::'a::foo)" and "Q (y::'a::bar)" -- "now illegal"
lemma "P (x::'a)" and "Q (y::'a::bar)"
- -- "now uniform 'a::bar instead of default sort for first occurence (!)"
+ -- "now uniform 'a::bar instead of default sort for first occurrence (!)"
*** HOL ***
--- a/README Sat Apr 14 12:36:11 2012 +0200
+++ b/README Sat Apr 14 12:46:45 2012 +0200
@@ -16,8 +16,8 @@
* The Poly/ML compiler and runtime system (version 5.2.1 or later).
* The GNU bash shell (version 3.x or 2.x).
* Perl (version 5.x).
- * Java 1.6.x from Oracle or Apple -- for Scala and jEdit.
- * GNU Emacs (version 23) -- for the Proof General 4.x interface.
+ * Java 1.6.x or 1.7.x from Oracle or Apple -- for Scala and jEdit.
+ * GNU Emacs (version 23 or 24) -- for the Proof General 4.x interface.
* A complete LaTeX installation -- for document preparation.
Installation