src/HOL/NSA/CLim.thy
changeset 57512 cc97b347b301
parent 56889 48a745e1bde7
child 57514 bdc2c6b40bf2
equal deleted inserted replaced
57511:de51a86fc903 57512:cc97b347b301
    20 
    20 
    21 text{*Changing the quantified variable. Install earlier?*}
    21 text{*Changing the quantified variable. Install earlier?*}
    22 lemma all_shift: "(\<forall>x::'a::comm_ring_1. P x) = (\<forall>x. P (x-a))";
    22 lemma all_shift: "(\<forall>x::'a::comm_ring_1. P x) = (\<forall>x. P (x-a))";
    23 apply auto 
    23 apply auto 
    24 apply (drule_tac x="x+a" in spec) 
    24 apply (drule_tac x="x+a" in spec) 
    25 apply (simp add: add_assoc) 
    25 apply (simp add: add.assoc) 
    26 done
    26 done
    27 
    27 
    28 lemma complex_add_minus_iff [simp]: "(x + - a = (0::complex)) = (x=a)"
    28 lemma complex_add_minus_iff [simp]: "(x + - a = (0::complex)) = (x=a)"
    29 by (simp add: diff_eq_eq)
    29 by (simp add: diff_eq_eq)
    30 
    30 
   140      "DERIV (%x. x ^ n) x :> (complex_of_real (real n)) * (x ^ (n - Suc 0))"
   140      "DERIV (%x. x ^ n) x :> (complex_of_real (real n)) * (x ^ (n - Suc 0))"
   141 apply (induct n)
   141 apply (induct n)
   142 apply (drule_tac [2] DERIV_ident [THEN DERIV_mult])
   142 apply (drule_tac [2] DERIV_ident [THEN DERIV_mult])
   143 apply (auto simp add: distrib_right real_of_nat_Suc)
   143 apply (auto simp add: distrib_right real_of_nat_Suc)
   144 apply (case_tac "n")
   144 apply (case_tac "n")
   145 apply (auto simp add: mult_ac add_commute)
   145 apply (auto simp add: mult_ac add.commute)
   146 done
   146 done
   147 
   147 
   148 text{*Nonstandard version*}
   148 text{*Nonstandard version*}
   149 lemma NSCDERIV_pow:
   149 lemma NSCDERIV_pow:
   150      "NSDERIV (%x. x ^ n) x :> complex_of_real (real n) * (x ^ (n - 1))"
   150      "NSDERIV (%x. x ^ n) x :> complex_of_real (real n) * (x ^ (n - 1))"