src/HOL/IMP/Hoare_Examples.thy
changeset 54489 03ff4d1e6784
parent 52554 19764bef2730
child 58410 6d46ad54a2ab
--- a/src/HOL/IMP/Hoare_Examples.thy	Tue Nov 19 01:30:14 2013 +0100
+++ b/src/HOL/IMP/Hoare_Examples.thy	Tue Nov 19 10:05:53 2013 +0100
@@ -2,17 +2,6 @@
 
 theory Hoare_Examples imports Hoare begin
 
-text{* Improves proof automation for negative numerals: *}
-
-lemma add_neg1R[simp]:
-  "x + -1 = x - (1 :: int)"
-by arith
-
-lemma add_neg_numeralR[simp]:
-  "x + neg_numeral n = (x::'a::neg_numeral) - numeral(n)"
-by (simp only: diff_minus_eq_add[symmetric] minus_neg_numeral)
-
-
 text{* Summing up the first @{text x} natural numbers in variable @{text y}. *}
 
 fun sum :: "int \<Rightarrow> int" where