src/HOL/Int.thy
changeset 59000 6eb0725503fc
parent 58889 5b7a9633cfa8
child 59536 03bde055a1a0
--- a/src/HOL/Int.thy	Thu Nov 13 14:40:06 2014 +0100
+++ b/src/HOL/Int.thy	Thu Nov 13 17:19:52 2014 +0100
@@ -493,7 +493,6 @@
 apply (rule_tac x="b - Suc a" in exI, arith)
 done
 
-
 subsection {* Cases and induction *}
 
 text{*Now we replace the case analysis rule by a more conventional one:
@@ -817,6 +816,12 @@
   with False show ?thesis by simp
 qed
 
+lemma nat_abs_int_diff: "nat \<bar>int a - int b\<bar> = (if a \<le> b then b - a else a - b)"
+  by auto
+
+lemma nat_int_add: "nat (int a + int b) = a + b"
+  by auto
+
 context ring_1
 begin