remove some redundant simp rules about sqrt
authorhuffman
Fri, 19 Aug 2011 19:01:00 -0700
changeset 44320 33439faadd67
parent 44319 806e0390de53
child 44321 975c9ba50a41
child 44327 46d5e7f52ba5
child 44342 8321948340ea
remove some redundant simp rules about sqrt
src/HOL/NthRoot.thy
--- a/src/HOL/NthRoot.thy	Fri Aug 19 18:42:41 2011 -0700
+++ b/src/HOL/NthRoot.thy	Fri Aug 19 19:01:00 2011 -0700
@@ -518,12 +518,6 @@
 apply (rule real_sqrt_abs)
 done
 
-lemma real_sqrt_pow2_gt_zero: "0 < x ==> 0 < (sqrt x)\<twosuperior>"
-by simp (* TODO: delete *)
-
-lemma real_sqrt_not_eq_zero: "0 < x ==> sqrt x \<noteq> 0"
-by simp (* TODO: delete *)
-
 lemma real_inv_sqrt_pow2: "0 < x ==> inverse (sqrt(x)) ^ 2 = inverse x"
 by (simp add: power_inverse [symmetric])
 
@@ -533,15 +527,6 @@
 lemma real_sqrt_ge_one: "1 \<le> x ==> 1 \<le> sqrt x"
 by simp
 
-lemma real_sqrt_two_gt_zero [simp]: "0 < sqrt 2"
-by simp
-
-lemma real_sqrt_two_ge_zero [simp]: "0 \<le> sqrt 2"
-by simp
-
-lemma real_sqrt_two_gt_one [simp]: "1 < sqrt 2"
-by simp
-
 lemma sqrt_divide_self_eq:
   assumes nneg: "0 \<le> x"
   shows "sqrt x / x = inverse (sqrt x)"
@@ -575,21 +560,18 @@
 
 subsection {* Square Root of Sum of Squares *}
 
-lemma real_sqrt_mult_self_sum_ge_zero [simp]: "0 \<le> sqrt(x*x + y*y)"
-by (rule real_sqrt_ge_zero [OF sum_squares_ge_zero])
-
-lemma real_sqrt_sum_squares_ge_zero [simp]: "0 \<le> sqrt (x\<twosuperior> + y\<twosuperior>)"
-by simp
+lemma real_sqrt_sum_squares_ge_zero: "0 \<le> sqrt (x\<twosuperior> + y\<twosuperior>)"
+  by simp (* TODO: delete *)
 
 declare real_sqrt_sum_squares_ge_zero [THEN abs_of_nonneg, simp]
 
 lemma real_sqrt_sum_squares_mult_ge_zero [simp]:
      "0 \<le> sqrt ((x\<twosuperior> + y\<twosuperior>)*(xa\<twosuperior> + ya\<twosuperior>))"
-by (auto intro!: real_sqrt_ge_zero simp add: zero_le_mult_iff)
+  by (simp add: zero_le_mult_iff)
 
 lemma real_sqrt_sum_squares_mult_squared_eq [simp]:
      "sqrt ((x\<twosuperior> + y\<twosuperior>) * (xa\<twosuperior> + ya\<twosuperior>)) ^ 2 = (x\<twosuperior> + y\<twosuperior>) * (xa\<twosuperior> + ya\<twosuperior>)"
-by (auto simp add: zero_le_mult_iff)
+  by (simp add: zero_le_mult_iff)
 
 lemma real_sqrt_sum_squares_eq_cancel: "sqrt (x\<twosuperior> + y\<twosuperior>) = x \<Longrightarrow> y = 0"
 by (drule_tac f = "%x. x\<twosuperior>" in arg_cong, simp)