src/HOL/Finite_Set.thy
changeset 32075 e8e0fb5da77a
parent 32006 0e209ff7f236
parent 32064 53ca12ff305d
child 32203 992ac8942691
--- a/src/HOL/Finite_Set.thy	Sat Jul 18 22:53:02 2009 +0200
+++ b/src/HOL/Finite_Set.thy	Mon Jul 20 08:32:07 2009 +0200
@@ -812,7 +812,7 @@
 by(rule fun_left_comm_idem.fold_insert_idem[OF ab_semigroup_idem_mult.fun_left_comm_idem[OF ab_semigroup_idem_mult_inf]])
 
 lemma inf_le_fold_inf: "finite A \<Longrightarrow> ALL a:A. b \<le> a \<Longrightarrow> inf b c \<le> fold inf c A"
-by (induct pred:finite) auto
+by (induct pred: finite) (auto intro: le_infI1)
 
 lemma fold_inf_le_inf: "finite A \<Longrightarrow> a \<in> A \<Longrightarrow> fold inf b A \<le> inf a b"
 proof(induct arbitrary: a pred:finite)
@@ -823,7 +823,7 @@
   proof cases
     assume "A = {}" thus ?thesis using insert by simp
   next
-    assume "A \<noteq> {}" thus ?thesis using insert by auto
+    assume "A \<noteq> {}" thus ?thesis using insert by (auto intro: le_infI2)
   qed
 qed