src/HOL/Complete_Lattice.thy
changeset 36635 080b755377c0
parent 36364 0e2679025aeb
child 37767 a2b7a20d6ea3
--- a/src/HOL/Complete_Lattice.thy	Tue May 04 08:55:39 2010 +0200
+++ b/src/HOL/Complete_Lattice.thy	Tue May 04 08:55:43 2010 +0200
@@ -33,8 +33,8 @@
 begin
 
 lemma dual_complete_lattice:
-  "complete_lattice Sup Inf (op \<ge>) (op >) (op \<squnion>) (op \<sqinter>) \<top> \<bottom>"
-  by (auto intro!: complete_lattice.intro dual_bounded_lattice)
+  "class.complete_lattice Sup Inf (op \<ge>) (op >) (op \<squnion>) (op \<sqinter>) \<top> \<bottom>"
+  by (auto intro!: class.complete_lattice.intro dual_bounded_lattice)
     (unfold_locales, (fact bot_least top_greatest
         Sup_upper Sup_least Inf_lower Inf_greatest)+)