diff -r 9207ada0ca31 -r f443ec10447d src/HOL/Library/Liminf_Limsup.thy --- a/src/HOL/Library/Liminf_Limsup.thy Thu Aug 30 19:59:36 2018 +0200 +++ b/src/HOL/Library/Liminf_Limsup.thy Thu Aug 30 17:20:54 2018 +0200 @@ -71,6 +71,11 @@ shows "(INF i : A. INF j : B. f i j) = (INF p : A \ B. f (fst p) (snd p))" by (rule antisym) (auto intro!: INF_greatest INF_lower2) +lemma INF_Sigma: + fixes f :: "_ \ _ \ _ :: complete_lattice" + shows "(INF i : A. INF j : B i. f i j) = (INF p : Sigma A B. f (fst p) (snd p))" + by (rule antisym) (auto intro!: INF_greatest INF_lower2) + subsubsection \\Liminf\ and \Limsup\\ definition Liminf :: "'a filter \ ('a \ 'b) \ 'b :: complete_lattice" where @@ -202,7 +207,7 @@ lemma le_Limsup: assumes F: "F \ bot" and x: "\\<^sub>F x in F. l \ f x" shows "l \ Limsup F f" - using F Liminf_bounded Liminf_le_Limsup order.trans x by blast + using F Liminf_bounded[of l f F] Liminf_le_Limsup[of F f] order.trans x by blast lemma Liminf_le: assumes F: "F \ bot" and x: "\\<^sub>F x in F. f x \ l"