src/HOL/Multivariate_Analysis/Extended_Real_Limits.thy
changeset 54258 adfc759263ab
parent 54257 5c7a3b6b05a9
child 54260 6a967667fd45
equal deleted inserted replaced
54257:5c7a3b6b05a9 54258:adfc759263ab
   658 proof -
   658 proof -
   659   {
   659   {
   660     assume "S \<noteq> {}"
   660     assume "S \<noteq> {}"
   661     { assume ex: "\<exists>B. \<forall>x\<in>S. B \<le> x"
   661     { assume ex: "\<exists>B. \<forall>x\<in>S. B \<le> x"
   662       then have *: "\<forall>x\<in>S. Inf S \<le> x"
   662       then have *: "\<forall>x\<in>S. Inf S \<le> x"
   663         using cInf_lower_EX[of _ S] ex by metis
   663         using cInf_lower[of _ S] ex by (metis bdd_below_def)
   664       then have "Inf S \<in> S"
   664       then have "Inf S \<in> S"
   665         apply (subst closed_contains_Inf)
   665         apply (subst closed_contains_Inf)
   666         using ex `S \<noteq> {}` `closed S`
   666         using ex `S \<noteq> {}` `closed S`
   667         apply auto
   667         apply auto
   668         done
   668         done