src/HOL/NthRoot.thy
changeset 78127 24b70433c2e8
parent 70722 ae2528273eeb
child 80175 200107cdd3ac
--- a/src/HOL/NthRoot.thy	Tue May 30 12:07:48 2023 +0200
+++ b/src/HOL/NthRoot.thy	Tue May 30 12:33:06 2023 +0100
@@ -460,10 +460,10 @@
 lemma real_sqrt_eq_iff [simp]: "sqrt x = sqrt y \<longleftrightarrow> x = y"
   unfolding sqrt_def by (rule real_root_eq_iff [OF pos2])
 
-lemma real_less_lsqrt: "0 \<le> x \<Longrightarrow> 0 \<le> y \<Longrightarrow> x < y\<^sup>2 \<Longrightarrow> sqrt x < y"
+lemma real_less_lsqrt: "0 \<le> y \<Longrightarrow> x < y\<^sup>2 \<Longrightarrow> sqrt x < y"
   using real_sqrt_less_iff[of x "y\<^sup>2"] by simp
 
-lemma real_le_lsqrt: "0 \<le> x \<Longrightarrow> 0 \<le> y \<Longrightarrow> x \<le> y\<^sup>2 \<Longrightarrow> sqrt x \<le> y"
+lemma real_le_lsqrt: "0 \<le> y \<Longrightarrow> x \<le> y\<^sup>2 \<Longrightarrow> sqrt x \<le> y"
   using real_sqrt_le_iff[of x "y\<^sup>2"] by simp
 
 lemma real_le_rsqrt: "x\<^sup>2 \<le> y \<Longrightarrow> x \<le> sqrt y"