src/HOL/Lattice/CompleteLattice.thy
changeset 11099 b301d1f72552
parent 10834 a7897aebbffc
child 11441 54b236801671
--- a/src/HOL/Lattice/CompleteLattice.thy	Sun Feb 11 20:38:40 2001 +0100
+++ b/src/HOL/Lattice/CompleteLattice.thy	Mon Feb 12 20:43:12 2001 +0100
@@ -16,7 +16,7 @@
   bounds (see \S\ref{sec:connect-bounds}).
 *}
 
-axclass complete_lattice < partial_order
+axclass complete_lattice \<subseteq> partial_order
   ex_Inf: "\<exists>inf. is_Inf A inf"
 
 theorem ex_Sup: "\<exists>sup::'a::complete_lattice. is_Sup A sup"
@@ -274,7 +274,7 @@
   thus ?thesis by (simp only: is_Sup_binary)
 qed
 
-instance complete_lattice < lattice
+instance complete_lattice \<subseteq> lattice
 proof
   fix x y :: "'a::complete_lattice"
   from is_inf_binary show "\<exists>inf. is_inf x y inf" ..