added lemma
authorhaftmann
Thu, 13 Dec 2007 07:09:00 +0100
changeset 25612 314d949c70b5
parent 25611 c0deb7307732
child 25613 bd055df900d3
added lemma
src/HOL/Nat.thy
--- a/src/HOL/Nat.thy	Thu Dec 13 07:08:59 2007 +0100
+++ b/src/HOL/Nat.thy	Thu Dec 13 07:09:00 2007 +0100
@@ -1443,6 +1443,13 @@
 text{*At present we prove no analogue of @{text not_less_Least} or @{text
 Least_Suc}, since there appears to be no need.*}
 
+text {* a nice rewrite for bounded subtraction *}
+
+lemma nat_minus_add_max:
+  fixes n m :: nat
+  shows "n - m + m = max n m"
+  by (simp add: max_def)
+
 
 subsection {*The Set of Natural Numbers*}