src/HOL/Library/Product_Lexorder.thy
changeset 54863 82acc20ded73
parent 53015 a1119cf551e8
child 58881 b9556a055632
--- a/src/HOL/Library/Product_Lexorder.thy	Wed Dec 25 17:39:06 2013 +0100
+++ b/src/HOL/Library/Product_Lexorder.thy	Wed Dec 25 17:39:06 2013 +0100
@@ -55,7 +55,7 @@
   "(sup :: 'a \<times> 'b \<Rightarrow> _ \<Rightarrow> _) = max"
 
 instance
-  by default (auto simp add: inf_prod_def sup_prod_def min_max.sup_inf_distrib1)
+  by default (auto simp add: inf_prod_def sup_prod_def max_min_distrib2)
 
 end