src/HOL/IMP/Abs_Int0.thy
changeset 52729 412c9e0381a1
parent 52504 52cd8bebc3b6
child 53015 a1119cf551e8
--- a/src/HOL/IMP/Abs_Int0.thy	Wed Jul 24 17:15:59 2013 +0200
+++ b/src/HOL/IMP/Abs_Int0.thy	Thu Jul 25 08:57:16 2013 +0200
@@ -6,11 +6,11 @@
 
 subsection "Orderings"
 
-text{* The basic type classes @{class order}, @{class semilattice_sup} and @{class top} are
+text{* The basic type classes @{class order}, @{class semilattice_sup} and @{class order_top} are
 defined in @{theory Main}, more precisely in theories @{theory Orderings} and @{theory Lattices}.
 If you view this theory with jedit, just click on the names to get there. *}
 
-class semilattice_sup_top = semilattice_sup + top
+class semilattice_sup_top = semilattice_sup + order_top
 
 
 instance "fun" :: (type, semilattice_sup_top) semilattice_sup_top ..
@@ -78,7 +78,7 @@
 lemma [simp]: "(Some x < Some y) = (x < y)"
 by(auto simp: less_le)
 
-instantiation option :: (order)bot
+instantiation option :: (order)order_bot
 begin
 
 definition bot_option :: "'a option" where