src/HOL/Lattices.thy
changeset 51546 2e26df807dc7
parent 51540 eea5c4ca4a0e
child 51593 d40aec502416
--- a/src/HOL/Lattices.thy	Tue Mar 26 20:55:21 2013 +0100
+++ b/src/HOL/Lattices.thy	Tue Mar 26 21:53:56 2013 +0100
@@ -471,25 +471,23 @@
 class bounded_semilattice_inf_top = semilattice_inf + top
 
 sublocale bounded_semilattice_inf_top < inf_top!: semilattice_neutr inf top
+  + inf_top!: semilattice_neutr_order inf top less_eq less
 proof
   fix x
   show "x \<sqinter> \<top> = x"
     by (rule inf_absorb1) simp
 qed
 
-sublocale bounded_semilattice_inf_top < inf_top!: semilattice_neutr_order inf top less_eq less ..
-
 class bounded_semilattice_sup_bot = semilattice_sup + bot
 
 sublocale bounded_semilattice_sup_bot < sup_bot!: semilattice_neutr sup bot
+  + sup_bot!: semilattice_neutr_order sup bot greater_eq greater
 proof
   fix x
   show "x \<squnion> \<bottom> = x"
     by (rule sup_absorb1) simp
 qed
 
-sublocale bounded_semilattice_sup_bot < sup_bot!: semilattice_neutr_order sup bot greater_eq greater ..
-
 class bounded_lattice_bot = lattice + bot
 begin