src/HOL/Finite_Set.thy
changeset 56166 9a241bc276cd
parent 56154 f0a927235162
child 56218 1c3f1f2431f9
--- a/src/HOL/Finite_Set.thy	Sat Mar 15 16:54:32 2014 +0100
+++ b/src/HOL/Finite_Set.thy	Sun Mar 16 18:09:04 2014 +0100
@@ -1041,7 +1041,7 @@
   interpret comp_fun_idem "inf \<circ> f" by (fact comp_comp_fun_idem)
   from `finite A` show "?fold = ?inf"
     by (induct A arbitrary: B)
-      (simp_all add: INF_def inf_left_commute)
+      (simp_all add: inf_left_commute)
 qed
 
 lemma sup_SUP_fold_sup:
@@ -1052,7 +1052,7 @@
   interpret comp_fun_idem "sup \<circ> f" by (fact comp_comp_fun_idem)
   from `finite A` show "?fold = ?sup"
     by (induct A arbitrary: B)
-      (simp_all add: SUP_def sup_left_commute)
+      (simp_all add: sup_left_commute)
 qed
 
 lemma INF_fold_inf: