added add_arith (just as hint by now)
authoroheimb
Tue, 20 Feb 2001 18:47:25 +0100
changeset 11164 03f5dc539fd9
parent 11163 14732e3eaa6e
child 11165 3b69feb7d053
added add_arith (just as hint by now)
src/HOL/NatArith.thy
--- a/src/HOL/NatArith.thy	Tue Feb 20 18:47:22 2001 +0100
+++ b/src/HOL/NatArith.thy	Tue Feb 20 18:47:25 2001 +0100
@@ -14,8 +14,14 @@
     "P(a - b::nat) = ((a<b --> P 0) & (ALL d. 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" *}
+ML {*
+ val nat_diff_split = thm "nat_diff_split";
+
+(* TODO: use this for force_tac in Provers/clasip.ML *)
+fun add_arith cs = cs addaltern ("arith_tac", arith_tac);
+*}
 
 lemmas [arith_split] = nat_diff_split split_min split_max
 
+
 end