Modified proofs for new hyp_subst_tac, and simplified them.
authorlcp
Thu, 06 Apr 1995 12:22:26 +0200
changeset 1020 76d72126a9e7
parent 1019 0697024c3cca
child 1021 9aa52d5d614f
Modified proofs for new hyp_subst_tac, and simplified them.
src/ZF/Coind/Map.ML
--- a/src/ZF/Coind/Map.ML	Thu Apr 06 12:20:48 1995 +0200
+++ b/src/ZF/Coind/Map.ML	Thu Apr 06 12:22:26 1995 +0200
@@ -50,7 +50,6 @@
 by (rtac subsetI 1);
 by (eresolve_tac prems 1);
 by (fast_tac ZF_cs 1);
-by flexflex_tac;
 qed "mapQU";
 
 (* ############################################################ *)
@@ -59,7 +58,6 @@
 
 goalw Map.thy [PMap_def,TMap_def] "!!A.B<=C ==> PMap(A,B)<=PMap(A,C)";
 by (fast_tac ZF_cs 1);
-by (flexflex_tac);
 qed "map_mono";
 
 (* Rename to pmap_mono *)
@@ -77,38 +75,23 @@
 
 (** map_owr **)
 
+
 goalw Map.thy [map_owr_def,PMap_def,TMap_def] 
   "!! A.[| m:PMap(A,B); a:A; b:B |]  ==> map_owr(m,a,b):PMap(A,B)";
 by (safe_tac ZF_cs);
-
-by (asm_full_simp_tac if_ss 1);
-by (fast_tac ZF_cs 1);
-
+by (asm_full_simp_tac if_ss 1 THEN fast_tac ZF_cs 1);
 by (fast_tac ZF_cs 1);
-
-by (rtac (excluded_middle RS disjE) 1);
-by (dtac (if_not_P RS subst) 1);
-by (assume_tac 1);
+by (asm_full_simp_tac (ZF_ss addsimps [if_iff]) 1);
 by (fast_tac ZF_cs 1);
-by (hyp_subst_tac 1);
-by (asm_full_simp_tac if_ss 1);
-by (fast_tac ZF_cs 1);
-
 by (rtac (excluded_middle RS disjE) 1);
 by (etac image_Sigma1 1);
-by (rtac (qbeta RS ssubst) 1);
-by (assume_tac 1);
-by (dtac map_lem1 1);
-by (etac qbeta 1);
-by (etac UnE'  1);
-by (etac singletonE 1);
-by (hyp_subst_tac 1);
-by (asm_full_simp_tac (if_ss addsimps [qbeta]) 1);
-by (etac notsingletonE 1);
-by (dtac map_lem1 1);
-by (rtac if_not_P 1);
-by (assume_tac 1);
-by (asm_full_simp_tac (if_ss addsimps [qbeta]) 1);
+by (safe_tac upair_cs);    (*This claset knows nothing about domain(m).*)
+by (asm_full_simp_tac (ZF_ss addsimps [qbeta]) 1);
+by (asm_simp_tac (ZF_ss addsimps [qbeta] setloop split_tac [expand_if]) 1);
+by (safe_tac FOL_cs);
+by (asm_full_simp_tac (ZF_ss addsimps [qbeta]) 1);
+by (dres_inst_tac [("psi", "?uu ~: B")] asm_rl 1);
+by (asm_full_simp_tac (ZF_ss addsimps [qbeta]) 1);
 by (fast_tac ZF_cs 1);
 qed "pmap_owrI";