src/HOL/NatArith.thy
changeset 17688 91d3604ec4b5
parent 17085 5b57f995a179
child 21238 c46bc715bdfd
--- a/src/HOL/NatArith.thy	Wed Sep 28 09:14:44 2005 +0200
+++ b/src/HOL/NatArith.thy	Wed Sep 28 11:14:26 2005 +0200
@@ -14,6 +14,9 @@
 
 text{*The following proofs may rely on the arithmetic proof procedures.*}
 
+lemma le_iff_add: "(m::nat) \<le> n = (\<exists>k. n = m + k)"
+  by (auto simp: le_eq_less_or_eq dest: less_imp_Suc_add)
+
 lemma pred_nat_trancl_eq_le: "((m, n) : pred_nat^*) = (m \<le> n)"
 by (simp add: less_eq reflcl_trancl [symmetric]
             del: reflcl_trancl, arith)