added addD2, addE2, addSD2, and addSE2
authoroheimb
Mon, 21 Sep 1998 23:06:37 +0200
changeset 5520 e2484f1786b7
parent 5519 54e313ed22ba
child 5521 7970832271cc
added addD2, addE2, addSD2, and addSE2 added not_Some_eq, also to simpset() and claset()
src/HOL/Option.ML
--- a/src/HOL/Option.ML	Mon Sep 21 23:04:51 1998 +0200
+++ b/src/HOL/Option.ML	Mon Sep 21 23:06:37 1998 +0200
@@ -11,6 +11,10 @@
 	(K [induct_tac "x" 1, Auto_tac]);
 AddIffs[not_None_eq];
 
+qed_goal "not_Some_eq" thy "(!y. x ~= Some y) = (x = None)"
+	(K [induct_tac "x" 1, Auto_tac]);
+AddIffs[not_Some_eq];
+
 
 section "case analysis in premises";
 
@@ -63,8 +67,8 @@
 
 qed_goal "ospec" thy 
 	"!!x. [| !x:o2s A. P x; A = Some x |] ==> P x" (K [Auto_tac]);
-claset_ref() := claset() addSaltern ("ospec", 
-				dmatch_tac [ospec] THEN' eq_assume_tac);
+AddDs[ospec];
+claset_ref() := claset() addSD2 ("ospec", ospec);
 
 
 val elem_o2s = prove_goal thy "!!X. x : o2s xo = (xo = Some x)"