src/HOL/Import/HOL_Light_Maps.thy
changeset 54863 82acc20ded73
parent 47364 637074507956
child 55393 ce5cebfaedda
--- a/src/HOL/Import/HOL_Light_Maps.thy	Wed Dec 25 17:39:06 2013 +0100
+++ b/src/HOL/Import/HOL_Light_Maps.thy	Wed Dec 25 17:39:06 2013 +0100
@@ -175,11 +175,11 @@
 
 lemma DEF_MAX[import_const "MAX"]:
   "max = (\<lambda>x y :: nat. if x \<le> y then y else x)"
-  by (auto simp add: min_max.le_iff_sup fun_eq_iff)
+  by (auto simp add: max.absorb_iff2 fun_eq_iff)
 
 lemma DEF_MIN[import_const "MIN"]:
   "min = (\<lambda>x y :: nat. if x \<le> y then x else y)"
-  by (auto simp add: min_max.le_iff_inf fun_eq_iff)
+  by (auto simp add: min.absorb_iff1 fun_eq_iff)
 
 lemma EVEN[import_const "EVEN" : "Parity.even_odd_class.even"]:
   "even (id 0\<Colon>nat) = True \<and> (\<forall>n. even (Suc n) = (\<not> even n))"