changeset 77140 | 9a60c1759543 |
parent 77138 | c8597292cd41 |
child 79566 | f783490c6c99 |
--- a/src/HOL/Power.thy Mon Jan 30 15:24:25 2023 +0000 +++ b/src/HOL/Power.thy Tue Jan 31 14:05:16 2023 +0000 @@ -89,6 +89,9 @@ lemma power4_eq_xxxx: "x^4 = x * x * x * x" by (simp add: mult.assoc power_numeral_even) +lemma power_numeral_reduce: "x ^ numeral n = x * x ^ pred_numeral n" + by (simp add: numeral_eq_Suc) + lemma funpow_times_power: "(times x ^^ f x) = times (x ^ f x)" proof (induct "f x" arbitrary: f) case 0