src/HOL/Multivariate_Analysis/Extended_Real_Limits.thy
changeset 61810 3c5040d5694a
parent 61560 7c985fd653c5
child 61973 0c7e865fa7cb
equal deleted inserted replaced
61809:81d34cf268d8 61810:3c5040d5694a
   429       by (intro complete_lattice_class.INF_lower) simp
   429       by (intro complete_lattice_class.INF_lower) simp
   430     with S have "f x \<in> S"
   430     with S have "f x \<in> S"
   431       by (simp add: mono_set)
   431       by (simp add: mono_set)
   432   }
   432   }
   433   with P show "eventually (\<lambda>x. f x \<in> S) net"
   433   with P show "eventually (\<lambda>x. f x \<in> S) net"
   434     by (auto elim: eventually_elim1)
   434     by (auto elim: eventually_mono)
   435 next
   435 next
   436   fix y l
   436   fix y l
   437   assume S: "\<forall>S. open S \<longrightarrow> mono_set S \<longrightarrow> l \<in> S \<longrightarrow> eventually  (\<lambda>x. f x \<in> S) net"
   437   assume S: "\<forall>S. open S \<longrightarrow> mono_set S \<longrightarrow> l \<in> S \<longrightarrow> eventually  (\<lambda>x. f x \<in> S) net"
   438   assume P: "\<forall>P. eventually P net \<longrightarrow> INFIMUM (Collect P) f \<le> y"
   438   assume P: "\<forall>P. eventually P net \<longrightarrow> INFIMUM (Collect P) f \<le> y"
   439   show "l \<le> y"
   439   show "l \<le> y"
   468       by (intro complete_lattice_class.SUP_upper) simp
   468       by (intro complete_lattice_class.SUP_upper) simp
   469     with S(1)[unfolded mono_set, rule_format, of "- SUPREMUM (Collect P) f" "- f x"] S(2)
   469     with S(1)[unfolded mono_set, rule_format, of "- SUPREMUM (Collect P) f" "- f x"] S(2)
   470     have "f x \<in> S"
   470     have "f x \<in> S"
   471       by (simp add: inj_image_mem_iff) }
   471       by (simp add: inj_image_mem_iff) }
   472   with P show "eventually (\<lambda>x. f x \<in> S) net"
   472   with P show "eventually (\<lambda>x. f x \<in> S) net"
   473     by (auto elim: eventually_elim1)
   473     by (auto elim: eventually_mono)
   474 next
   474 next
   475   fix y l
   475   fix y l
   476   assume S: "\<forall>S. open S \<longrightarrow> mono_set (uminus ` S) \<longrightarrow> l \<in> S \<longrightarrow> eventually  (\<lambda>x. f x \<in> S) net"
   476   assume S: "\<forall>S. open S \<longrightarrow> mono_set (uminus ` S) \<longrightarrow> l \<in> S \<longrightarrow> eventually  (\<lambda>x. f x \<in> S) net"
   477   assume P: "\<forall>P. eventually P net \<longrightarrow> y \<le> SUPREMUM (Collect P) f"
   477   assume P: "\<forall>P. eventually P net \<longrightarrow> y \<le> SUPREMUM (Collect P) f"
   478   show "y \<le> l"
   478   show "y \<le> l"