src/HOL/Library/Saturated.thy
changeset 51540 eea5c4ca4a0e
parent 51489 f738e6dbd844
child 51545 6f6012f430fc
--- a/src/HOL/Library/Saturated.thy	Tue Mar 26 15:10:28 2013 +0100
+++ b/src/HOL/Library/Saturated.thy	Tue Mar 26 20:49:57 2013 +0100
@@ -45,7 +45,7 @@
 
 lemma min_nat_of_len_of [simp]:
   "min (nat_of (n::('a::len) sat)) (len_of TYPE('a)) = nat_of n"
-  by (subst min_max.inf.commute) simp
+  by (subst min.commute) simp
 
 lemma Abs_sat'_nat_of [simp]:
   "Abs_sat' (nat_of n) = n"