remove redundant lemmas
authorhuffman
Mon, 14 May 2007 09:27:24 +0200
changeset 22961 e499ded5d0fc
parent 22960 114cf1906681
child 22962 4bb05ba38939
remove redundant lemmas
src/HOL/Hyperreal/NthRoot.thy
--- a/src/HOL/Hyperreal/NthRoot.thy	Mon May 14 09:16:47 2007 +0200
+++ b/src/HOL/Hyperreal/NthRoot.thy	Mon May 14 09:27:24 2007 +0200
@@ -474,14 +474,11 @@
 
 subsection {* Square Root of Sum of Squares *}
 
-lemma "(sqrt (x\<twosuperior> + y\<twosuperior>))\<twosuperior> = x\<twosuperior> + y\<twosuperior>"
-by simp
-
 lemma real_sqrt_mult_self_sum_ge_zero [simp]: "0 \<le> sqrt(x*x + y*y)"
-by (rule real_sqrt_ge_zero [OF real_mult_self_sum_ge_zero]) 
+by (rule real_sqrt_ge_zero [OF real_mult_self_sum_ge_zero])
 
 lemma real_sqrt_sum_squares_ge_zero [simp]: "0 \<le> sqrt (x\<twosuperior> + y\<twosuperior>)"
-by (auto intro!: real_sqrt_ge_zero)
+by simp
 
 lemma real_sqrt_sum_squares_mult_ge_zero [simp]:
      "0 \<le> sqrt ((x\<twosuperior> + y\<twosuperior>)*(xa\<twosuperior> + ya\<twosuperior>))"
@@ -497,12 +494,6 @@
 lemma real_sqrt_sum_squares_ge2 [simp]: "y \<le> sqrt(x\<twosuperior> + y\<twosuperior>)"
 by (rule power2_le_imp_le, simp_all)
 
-lemma real_sqrt_sos_less_one_iff: "(sqrt (x\<twosuperior> + y\<twosuperior>) < 1) = (x\<twosuperior> + y\<twosuperior> < 1)"
-by (rule real_sqrt_lt_1_iff)
-
-lemma real_sqrt_sos_eq_one_iff: "(sqrt (x\<twosuperior> + y\<twosuperior>) = 1) = (x\<twosuperior> + y\<twosuperior> = 1)"
-by (rule real_sqrt_eq_1_iff)
-
 lemma power2_sum:
   fixes x y :: "'a::{number_ring,recpower}"
   shows "(x + y)\<twosuperior> = x\<twosuperior> + y\<twosuperior> + 2 * x * y"