diff -r 217bececa2bd -r bb6f072c8d10 src/HOL/Real/RealPow.thy --- a/src/HOL/Real/RealPow.thy Mon Oct 18 13:40:45 2004 +0200 +++ b/src/HOL/Real/RealPow.thy Tue Oct 19 18:18:45 2004 +0200 @@ -57,7 +57,7 @@ by (insert power_increasing [of 0 n "2::real"], simp) lemma two_realpow_gt [simp]: "real (n::nat) < 2 ^ n" -apply (induct_tac "n") +apply (induct "n") apply (auto simp add: real_of_nat_Suc) apply (subst mult_2) apply (rule real_add_less_le_mono) @@ -97,12 +97,12 @@ done lemma realpow_real_of_nat: "real (m::nat) ^ n = real (m ^ n)" -apply (induct_tac "n") +apply (induct "n") apply (auto simp add: real_of_nat_one real_of_nat_mult) done lemma realpow_real_of_nat_two_pos [simp] : "0 < real (Suc (Suc 0) ^ n)" -apply (induct_tac "n") +apply (induct "n") apply (auto simp add: real_of_nat_mult zero_less_mult_iff) done @@ -113,12 +113,12 @@ lemma zero_less_realpow_abs_iff [simp]: "(0 < (abs x)^n) = (x \ (0::real) | n=0)" -apply (induct_tac "n") +apply (induct "n") apply (auto simp add: zero_less_mult_iff) done lemma zero_le_realpow_abs [simp]: "(0::real) \ (abs x)^n" -apply (induct_tac "n") +apply (induct "n") apply (auto simp add: zero_le_mult_iff) done @@ -126,7 +126,7 @@ subsection{*Literal Arithmetic Involving Powers, Type @{typ real}*} lemma real_of_int_power: "real (x::int) ^ n = real (x ^ n)" -apply (induct_tac "n") +apply (induct "n") apply (simp_all add: nat_mult_distrib) done declare real_of_int_power [symmetric, simp] @@ -235,7 +235,7 @@ by (case_tac "n", auto) lemma real_num_zero_less_two_pow [simp]: "0 < (2::real) ^ (4*d)" -apply (induct_tac "d") +apply (induct "d") apply (auto simp add: realpow_num_eq_if) done