src/HOL/Library/Nonpos_Ints.thy
changeset 67135 1a94352812f4
parent 63092 a949b2a5f51d
child 68499 d4312962161a
--- a/src/HOL/Library/Nonpos_Ints.thy	Mon Dec 04 23:10:52 2017 +0100
+++ b/src/HOL/Library/Nonpos_Ints.thy	Tue Dec 05 12:14:36 2017 +0100
@@ -1,4 +1,4 @@
-(*  Title:    HOL/Library/Nonpos_Ints.thy
+  (*  Title:    HOL/Library/Nonpos_Ints.thy
     Author:   Manuel Eberl, TU München
 *)
 
@@ -237,7 +237,6 @@
 lemma uminus_nonneg_Reals_iff [simp]: "-x \<in> \<real>\<^sub>\<ge>\<^sub>0 \<longleftrightarrow> x \<in> \<real>\<^sub>\<le>\<^sub>0"
   apply (auto simp: nonpos_Reals_def nonneg_Reals_def)
   apply (metis nonpos_Reals_of_real_iff minus_minus neg_le_0_iff_le of_real_minus)
-  apply (metis neg_0_le_iff_le of_real_minus)
   done
 
 lemma uminus_nonpos_Reals_iff [simp]: "-x \<in> \<real>\<^sub>\<le>\<^sub>0 \<longleftrightarrow> x \<in> \<real>\<^sub>\<ge>\<^sub>0"