src/HOL/Analysis/Complex_Transcendental.thy
changeset 82861 3e1521dc095d
parent 82860 0b38dccd8cf5
child 82882 253db0f4c540
--- a/src/HOL/Analysis/Complex_Transcendental.thy	Mon Jul 14 12:33:34 2025 +0100
+++ b/src/HOL/Analysis/Complex_Transcendental.thy	Mon Jul 14 18:41:41 2025 +0100
@@ -2465,6 +2465,7 @@
 lemma complex_powr_of_int: "z \<noteq> 0 \<or> n \<noteq> 0 \<Longrightarrow> z powr of_int n = (z :: complex) powi n"
   by (cases "z = 0 \<or> n = 0")
      (auto simp: power_int_def powr_minus powr_nat powr_of_int power_0_left power_inverse)
+
 lemma powr_of_neg_real:
   fixes x::real and y::real
   assumes "x<0"