deleted redundant theorem
authorpaulson <lp15@cam.ac.uk>
Tue, 26 Jun 2018 15:44:35 +0100
changeset 68501 8a8f98c84df3
parent 68500 e3e742b9eed4
child 68502 a8ada04583e7
deleted redundant theorem
src/HOL/Nonstandard_Analysis/NSA.thy
--- a/src/HOL/Nonstandard_Analysis/NSA.thy	Tue Jun 26 14:51:32 2018 +0100
+++ b/src/HOL/Nonstandard_Analysis/NSA.thy	Tue Jun 26 15:44:35 2018 +0100
@@ -132,12 +132,6 @@
 
 subsection \<open>Closure Laws for the Standard Reals\<close>
 
-lemma Reals_minus_iff [simp]: "- x \<in> \<real> \<longleftrightarrow> x \<in> \<real>"
-  apply auto
-  apply (drule Reals_minus)
-  apply auto
-  done
-
 lemma Reals_add_cancel: "x + y \<in> \<real> \<Longrightarrow> y \<in> \<real> \<Longrightarrow> x \<in> \<real>"
   by (drule (1) Reals_diff) simp