src/HOL/List.thy
changeset 54498 f7fef6b00bfe
parent 54496 178922b63b58
parent 54489 03ff4d1e6784
child 54555 e8c5e95d338b
child 54593 8c0a27b9c1bd
--- a/src/HOL/List.thy	Mon Nov 18 17:15:01 2013 +0100
+++ b/src/HOL/List.thy	Tue Nov 19 17:07:52 2013 +0100
@@ -3075,9 +3075,9 @@
 
 lemmas upto_rec_numeral [simp] =
   upto.simps[of "numeral m" "numeral n"]
-  upto.simps[of "numeral m" "neg_numeral n"]
-  upto.simps[of "neg_numeral m" "numeral n"]
-  upto.simps[of "neg_numeral m" "neg_numeral n"] for m n
+  upto.simps[of "numeral m" "- numeral n"]
+  upto.simps[of "- numeral m" "numeral n"]
+  upto.simps[of "- numeral m" "- numeral n"] for m n
 
 lemma upto_empty[simp]: "j < i \<Longrightarrow> [i..j] = []"
 by(simp add: upto.simps)