src/HOL/Hyperreal/HTranscendental.thy
changeset 20217 25b068a99d2b
parent 19765 dfe940911617
child 20552 2c31dd358c21
equal deleted inserted replaced
20216:f30b73385060 20217:25b068a99d2b
   362 lemma starfun_exp_HFinite: "x \<in> HFinite ==> ( *f* exp) x \<in> HFinite"
   362 lemma starfun_exp_HFinite: "x \<in> HFinite ==> ( *f* exp) x \<in> HFinite"
   363 apply (cases x)
   363 apply (cases x)
   364 apply (auto simp add: starfun HFinite_FreeUltrafilterNat_iff)
   364 apply (auto simp add: starfun HFinite_FreeUltrafilterNat_iff)
   365 apply (rule bexI [OF _ Rep_star_star_n], auto)
   365 apply (rule bexI [OF _ Rep_star_star_n], auto)
   366 apply (rule_tac x = "exp u" in exI)
   366 apply (rule_tac x = "exp u" in exI)
   367 apply (ultra, arith)
   367 apply ultra
   368 done
   368 done
   369 
   369 
   370 lemma starfun_exp_add_HFinite_Infinitesimal_approx:
   370 lemma starfun_exp_add_HFinite_Infinitesimal_approx:
   371      "[|x \<in> Infinitesimal; z \<in> HFinite |] ==> ( *f* exp) (z + x) @= ( *f* exp) z"
   371      "[|x \<in> Infinitesimal; z \<in> HFinite |] ==> ( *f* exp) (z + x) @= ( *f* exp) z"
   372 apply (simp add: STAR_exp_add)
   372 apply (simp add: STAR_exp_add)