redundant: dropped
authorhaftmann
Thu, 02 Oct 2014 11:33:05 +0200
changeset 58511 97aec08d6f28
parent 58510 c6427c9d0898
child 58512 dc4d76dfa8f0
redundant: dropped
src/HOL/Divides.thy
--- a/src/HOL/Divides.thy	Thu Oct 02 11:33:04 2014 +0200
+++ b/src/HOL/Divides.thy	Thu Oct 02 11:33:05 2014 +0200
@@ -2425,16 +2425,6 @@
 
 subsubsection {* The Divides Relation *}
 
-lemma dvd_neg_numeral_left [simp]:
-  fixes y :: "'a::comm_ring_1"
-  shows "(- numeral k) dvd y \<longleftrightarrow> (numeral k) dvd y"
-  by (fact minus_dvd_iff)
-
-lemma dvd_neg_numeral_right [simp]:
-  fixes x :: "'a::comm_ring_1"
-  shows "x dvd (- numeral k) \<longleftrightarrow> x dvd (numeral k)"
-  by (fact dvd_minus_iff)
-
 lemmas dvd_eq_mod_eq_0_numeral [simp] =
   dvd_eq_mod_eq_0 [of "numeral x" "numeral y"] for x y