src/HOL/Decision_Procs/Approximation.thy
changeset 56382 5a50109d51ab
parent 56381 0556204bc230
child 56410 a14831ac3023
equal deleted inserted replaced
56381:0556204bc230 56382:5a50109d51ab
  2676   thus ?case
  2676   thus ?case
  2677     by (auto intro!: derivative_eq_intros simp add: algebra_simps power2_eq_square)
  2677     by (auto intro!: derivative_eq_intros simp add: algebra_simps power2_eq_square)
  2678 next
  2678 next
  2679   case (Cos a)
  2679   case (Cos a)
  2680   thus ?case
  2680   thus ?case
  2681     by (auto intro!: derivative_intros
  2681     by (auto intro!: derivative_eq_intros
  2682            simp del: interpret_floatarith.simps(5)
  2682            simp del: interpret_floatarith.simps(5)
  2683            simp add: interpret_floatarith_sin interpret_floatarith.simps(5)[of a])
  2683            simp add: interpret_floatarith_sin interpret_floatarith.simps(5)[of a])
  2684 next
  2684 next
  2685   case (Power a n)
  2685   case (Power a n)
  2686   thus ?case
  2686   thus ?case
  2687     by (cases n) (auto intro!: derivative_intros simp del: power_Suc)
  2687     by (cases n) (auto intro!: derivative_eq_intros simp del: power_Suc simp add: real_of_nat_def)
  2688 next
  2688 next
  2689   case (Ln a)
  2689   case (Ln a)
  2690   thus ?case by (auto intro!: derivative_intros simp add: divide_inverse)
  2690   thus ?case by (auto intro!: derivative_eq_intros simp add: divide_inverse)
  2691 next
  2691 next
  2692   case (Var i)
  2692   case (Var i)
  2693   thus ?case using `n < length vs` by auto
  2693   thus ?case using `n < length vs` by auto
  2694 qed (auto intro!: derivative_eq_intros)
  2694 qed (auto intro!: derivative_eq_intros)
  2695 
  2695