src/HOL/IMP/Abs_Int0.thy
changeset 51625 bd3358aac5d2
parent 51390 1dff81cf425b
child 51628 0a6d576da295
--- a/src/HOL/IMP/Abs_Int0.thy	Fri Apr 05 15:13:25 2013 +0200
+++ b/src/HOL/IMP/Abs_Int0.thy	Fri Apr 05 18:31:35 2013 +0200
@@ -6,7 +6,9 @@
 
 subsection "Orderings"
 
-declare order_trans[trans]
+text{* The basic type classes @{class order}, @{class semilattice_sup} and @{class 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 = semilattice_sup + top