NEWS
changeset 67831 07f5588f2735
parent 67830 4f992daf4707
child 67904 465f43a9f780
--- a/NEWS	Mon Mar 12 20:53:29 2018 +0100
+++ b/NEWS	Mon Mar 12 21:03:57 2018 +0100
@@ -9,16 +9,6 @@
 
 *** General ***
 
-* New, more general, axiomatization of complete_distrib_lattice. 
-The former axioms:
-"sup x (Inf X) = Inf (sup x ` X)" and "inf x (Sup X) = Sup (inf x ` X)"
-are replaced by 
-"Inf (Sup ` A) <= Sup (Inf ` {f ` A | f . (! Y \<in> A . f Y \<in> Y)})"
-The instantiations of sets and functions as complete_distrib_lattice 
-are moved to Hilbert_Choice.thy because their proofs need the Hilbert
-choice operator. The dual of this property is also proved in 
-Hilbert_Choice.thy.
-
 * Marginal comments need to be written exclusively in the new-style form
 "\<comment> \<open>text\<close>", old ASCII variants like "-- {* ... *}" are no longer
 supported. INCOMPATIBILITY, use the command-line tool "isabelle
@@ -204,6 +194,16 @@
 
 *** HOL ***
 
+* New, more general, axiomatization of complete_distrib_lattice. 
+The former axioms:
+"sup x (Inf X) = Inf (sup x ` X)" and "inf x (Sup X) = Sup (inf x ` X)"
+are replaced by 
+"Inf (Sup ` A) <= Sup (Inf ` {f ` A | f . (! Y \<in> A . f Y \<in> Y)})"
+The instantiations of sets and functions as complete_distrib_lattice 
+are moved to Hilbert_Choice.thy because their proofs need the Hilbert
+choice operator. The dual of this property is also proved in 
+Hilbert_Choice.thy.
+
 * Clarifed theorem names:
 
   Min.antimono ~> Min.subset_imp