src/HOL/Transcendental.thy
changeset 77490 2c86ea8961b5
parent 77230 2d26af072990
child 78250 400aecdfd71f
--- a/src/HOL/Transcendental.thy	Thu Mar 02 11:34:54 2023 +0000
+++ b/src/HOL/Transcendental.thy	Thu Mar 02 17:17:18 2023 +0000
@@ -2492,6 +2492,9 @@
       for a x :: "'a::{ln,real_normed_field}"
   by (simp add: divide_inverse powr_minus)
 
+lemma powr_sum: "x \<noteq> 0 \<Longrightarrow> finite A \<Longrightarrow> x powr sum f A = (\<Prod>y\<in>A. x powr f y)"
+  by (simp add: powr_def exp_sum sum_distrib_right)
+
 lemma divide_powr_uminus: "a / b powr c = a * b powr (- c)"
   for a b c :: real
   by (simp add: powr_minus_divide)