src/HOL/Lattices_Big.thy
changeset 54863 82acc20ded73
parent 54857 5c05f7c5f8ae
child 54864 a064732223ad
--- a/src/HOL/Lattices_Big.thy	Wed Dec 25 17:39:06 2013 +0100
+++ b/src/HOL/Lattices_Big.thy	Wed Dec 25 17:39:06 2013 +0100
@@ -371,10 +371,10 @@
     by (simp only: min_max.Sup_fin_def Max_def)
 qed
 
-lemmas le_maxI1 = min_max.sup_ge1
-lemmas le_maxI2 = min_max.sup_ge2
-lemmas min_ac = min.assoc min_max.inf_commute min.left_commute
-lemmas max_ac = min_max.sup_assoc min_max.sup_commute max.left_commute
+lemmas le_maxI1 = max.cobounded1
+lemmas le_maxI2 = max.cobounded2
+lemmas min_ac = min.assoc min.commute min.left_commute
+lemmas max_ac = max.assoc max.commute max.left_commute
 
 end