src/HOL/Hyperreal/HTranscendental.thy
changeset 27148 5b78e50adc49
parent 23177 3004310c95b1
equal deleted inserted replaced
27147:62ab1968c1f4 27148:5b78e50adc49
   304 done
   304 done
   305 
   305 
   306 lemma starfun_exp_gt_one [simp]: "!!x::hypreal. 0 < x ==> 1 < ( *f* exp) x"
   306 lemma starfun_exp_gt_one [simp]: "!!x::hypreal. 0 < x ==> 1 < ( *f* exp) x"
   307 by transfer (rule exp_gt_one)
   307 by transfer (rule exp_gt_one)
   308 
   308 
   309 (* needs derivative of inverse function
       
   310    TRY a NS one today!!!
       
   311 
       
   312 Goal "x @= 1 ==> ( *f* ln) x @= 1"
       
   313 by (res_inst_tac [("z","x")] eq_Abs_star 1);
       
   314 by (auto_tac (claset(),simpset() addsimps [hypreal_one_def]));
       
   315 
       
   316 
       
   317 Goalw [nsderiv_def] "0r < x ==> NSDERIV ln x :> inverse x";
       
   318 
       
   319 *)
       
   320 
       
   321 
       
   322 lemma starfun_ln_exp [simp]: "!!x. ( *f* ln) (( *f* exp) x) = x"
   309 lemma starfun_ln_exp [simp]: "!!x. ( *f* ln) (( *f* exp) x) = x"
   323 by transfer (rule ln_exp)
   310 by transfer (rule ln_exp)
   324 
   311 
   325 lemma starfun_exp_ln_iff [simp]: "!!x. (( *f* exp)(( *f* ln) x) = x) = (0 < x)"
   312 lemma starfun_exp_ln_iff [simp]: "!!x. (( *f* exp)(( *f* ln) x) = x) = (0 < x)"
   326 by transfer (rule exp_ln_iff)
   313 by transfer (rule exp_ln_iff)