src/HOL/NatArith.thy
changeset 10214 77349ed89f45
child 10599 2df753cf86e9
--- /dev/null	Thu Jan 01 00:00:00 1970 +0000
+++ b/src/HOL/NatArith.thy	Fri Oct 13 08:28:21 2000 +0200
@@ -0,0 +1,21 @@
+(*  Title:      HOL/NatArith.thy
+    ID:         $Id$
+
+Setup arithmetic proof procedures.
+*)
+
+theory NatArith = Nat
+files "arith_data.ML":
+
+setup arith_setup
+
+(*elimination of `-' on nat*)
+lemma nat_diff_split:
+    "P(a - b::nat) = (ALL d. (a<b --> P 0) & (a = b + d --> P d))"
+  by (cases "a < b" rule: case_split) (auto simp add: diff_is_0_eq [THEN iffD2])
+
+ML {* val nat_diff_split = thm "nat_diff_split" *}
+
+lemmas [arith_split] = nat_diff_split split_min split_max
+
+end