src/HOL/Filter.thy
changeset 62378 85ed00c1fe7c
parent 62369 acfc4ad7b76a
child 62379 340738057c8c
--- a/src/HOL/Filter.thy	Fri Feb 12 16:09:07 2016 +0100
+++ b/src/HOL/Filter.thy	Fri Feb 19 13:40:50 2016 +0100
@@ -490,7 +490,7 @@
   shows "\<forall>\<^sub>F x in \<Sqinter>i\<in>I. F' i. T P x"
 proof -
   from * obtain X where "finite X" "X \<subseteq> I" "\<forall>\<^sub>F x in \<Sqinter>i\<in>X. F i. P x"
-    unfolding eventually_INF[of _ I] by auto
+    unfolding eventually_INF[of _ _ I] by auto
   moreover then have "eventually (T P) (INFIMUM X F')"
     apply (induction X arbitrary: P)
     apply (auto simp: eventually_inf T2)