src/HOL/Lattices_Big.thy
changeset 54857 5c05f7c5f8ae
parent 54745 46e441e61ff5
child 54863 82acc20ded73
--- a/src/HOL/Lattices_Big.thy	Tue Dec 24 11:24:14 2013 +0100
+++ b/src/HOL/Lattices_Big.thy	Tue Dec 24 11:24:16 2013 +0100
@@ -373,12 +373,8 @@
 
 lemmas le_maxI1 = min_max.sup_ge1
 lemmas le_maxI2 = min_max.sup_ge2
- 
-lemmas min_ac = min_max.inf_assoc min_max.inf_commute
-  min.left_commute
-
-lemmas max_ac = min_max.sup_assoc min_max.sup_commute
-  max.left_commute
+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
 
 end