src/HOL/Nonstandard_Analysis/HLim.thy
changeset 63040 eb4ddd18d635
parent 62479 716336f19aa9
child 63579 73939a9b70a3
equal deleted inserted replaced
63039:1a20fd9cf281 63040:eb4ddd18d635
   207 apply (simp add: isNSCont_def NSLIM_def, auto)
   207 apply (simp add: isNSCont_def NSLIM_def, auto)
   208 apply (case_tac "y = star_of a", auto)
   208 apply (case_tac "y = star_of a", auto)
   209 done
   209 done
   210 
   210 
   211 text\<open>NS continuity can be defined using NS Limit in
   211 text\<open>NS continuity can be defined using NS Limit in
   212     similar fashion to standard def of continuity\<close>
   212     similar fashion to standard definition of continuity\<close>
   213 lemma isNSCont_NSLIM_iff: "(isNSCont f a) = (f \<midarrow>a\<rightarrow>\<^sub>N\<^sub>S (f a))"
   213 lemma isNSCont_NSLIM_iff: "(isNSCont f a) = (f \<midarrow>a\<rightarrow>\<^sub>N\<^sub>S (f a))"
   214 by (blast intro: isNSCont_NSLIM NSLIM_isNSCont)
   214 by (blast intro: isNSCont_NSLIM NSLIM_isNSCont)
   215 
   215 
   216 text\<open>Hence, NS continuity can be given
   216 text\<open>Hence, NS continuity can be given
   217   in terms of standard limit\<close>
   217   in terms of standard limit\<close>
   234 by (erule isNSCont_isCont_iff [THEN iffD1])
   234 by (erule isNSCont_isCont_iff [THEN iffD1])
   235 
   235 
   236 text\<open>Alternative definition of continuity\<close>
   236 text\<open>Alternative definition of continuity\<close>
   237 
   237 
   238 (* Prove equivalence between NS limits - *)
   238 (* Prove equivalence between NS limits - *)
   239 (* seems easier than using standard def  *)
   239 (* seems easier than using standard definition  *)
   240 lemma NSLIM_h_iff: "(f \<midarrow>a\<rightarrow>\<^sub>N\<^sub>S L) = ((%h. f(a + h)) \<midarrow>0\<rightarrow>\<^sub>N\<^sub>S L)"
   240 lemma NSLIM_h_iff: "(f \<midarrow>a\<rightarrow>\<^sub>N\<^sub>S L) = ((%h. f(a + h)) \<midarrow>0\<rightarrow>\<^sub>N\<^sub>S L)"
   241 apply (simp add: NSLIM_def, auto)
   241 apply (simp add: NSLIM_def, auto)
   242 apply (drule_tac x = "star_of a + x" in spec)
   242 apply (drule_tac x = "star_of a + x" in spec)
   243 apply (drule_tac [2] x = "- star_of a + x" in spec, safe, simp)
   243 apply (drule_tac [2] x = "- star_of a + x" in spec, safe, simp)
   244 apply (erule mem_infmal_iff [THEN iffD2, THEN Infinitesimal_add_approx_self [THEN approx_sym]])
   244 apply (erule mem_infmal_iff [THEN iffD2, THEN Infinitesimal_add_approx_self [THEN approx_sym]])