changeset 65057 | 799bbbb3a395 |
parent 64964 | a0c985a57f7e |
child 66912 | a99a7cbf0fb5 |
--- a/src/HOL/Power.thy Mon Feb 27 00:00:28 2017 +0100 +++ b/src/HOL/Power.thy Mon Feb 27 17:17:26 2017 +0000 @@ -563,6 +563,11 @@ lemma power_Suc_le_self: "0 \<le> a \<Longrightarrow> a \<le> 1 \<Longrightarrow> a ^ Suc n \<le> a" using power_decreasing [of 1 "Suc n" a] by simp +lemma power2_eq_iff_nonneg [simp]: + assumes "0 \<le> x" "0 \<le> y" + shows "(x ^ 2 = y ^ 2) \<longleftrightarrow> x = y" +using assms power2_eq_imp_eq by blast + end context linordered_ring_strict