src/ZF/Resid/Cube.ML
changeset 5527 38928c4a8eb2
parent 5147 825877190618
child 6046 2c8a8be36c94
--- a/src/ZF/Resid/Cube.ML	Mon Sep 21 23:25:27 1998 +0200
+++ b/src/ZF/Resid/Cube.ML	Tue Sep 22 13:48:32 1998 +0200
@@ -7,9 +7,8 @@
 
 open Cube;
 
-val prism_ss = (res1L_ss addsimps 
-                [commutation,residuals_preserve_comp,sub_preserve_reg,
-                 residuals_preserve_reg,sub_comp,sub_comp RS comp_sym]);
+Addsimps [commutation, residuals_preserve_comp, sub_preserve_reg,
+	  residuals_preserve_reg, sub_comp, sub_comp RS comp_sym];
 
 (* ------------------------------------------------------------------------- *)
 (*         Prism theorem                                                     *)
@@ -18,24 +17,17 @@
 
 (* Having more assumptions than needed -- removed below  *)
 Goal "v<==u ==> \
-\   regular(u)-->(ALL w. w~v-->w~u-->  \
-\             w |> u = (w|>v) |> (u|>v))";
+\   regular(u) --> (ALL w. w~v --> w~u -->  \
+\                          w |> u = (w|>v) |> (u|>v))";
 by (etac Ssub.induct 1);
-by (ALLGOALS (asm_simp_tac prism_ss));
-by (dresolve_tac [spec RS mp RS mp] 1 THEN resolve_tac [Scomp.Comp_Fun] 1 
-    THEN resolve_tac [Scomp.Comp_Fun] 2 THEN (REPEAT(assume_tac 1)));
-by (asm_full_simp_tac prism_ss 1);
-by (dresolve_tac [spec RS mp RS mp] 1 THEN resolve_tac [Scomp.Comp_Fun] 1 
-    THEN resolve_tac [Scomp.Comp_Fun] 2 THEN (REPEAT(assume_tac 1)));
-by (asm_full_simp_tac prism_ss 1);
+by Auto_tac;
 qed_spec_mp "prism_l";
 
 Goal "[|v <== u; regular(u); w~v|]==> \
 \       w |> u = (w|>v) |> (u|>v)";
 by (rtac prism_l 1);
 by (rtac comp_trans 4);
-by (assume_tac 4);
-by (ALLGOALS(asm_simp_tac prism_ss));
+by Auto_tac;
 qed "prism";
 
 
@@ -53,9 +45,9 @@
 by (asm_full_simp_tac (simpset() addsimps 
 		       [prism RS sym,union_l,union_preserve_regular,
 			comp_sym_iff, union_sym]) 4);
-by (asm_full_simp_tac (simpset() addsimps [union_r, comp_sym_iff]) 1);
-by (asm_full_simp_tac (simpset() addsimps 
-		       [union_preserve_regular, comp_sym_iff]) 1);
+by (asm_simp_tac (simpset() addsimps [union_r, comp_sym_iff]) 1);
+by (asm_simp_tac (simpset() addsimps 
+		  [union_preserve_regular, comp_sym_iff]) 1);
 by (etac comp_trans 1);
 by (atac 1);
 qed "cube";
@@ -71,7 +63,7 @@
 by (subgoal_tac "u~v" 1);
 by (safe_tac (claset() addSIs [exI]));
 by (rtac cube 1);
-by (ALLGOALS (asm_simp_tac (prism_ss addsimps [comp_sym_iff])));
+by (ALLGOALS (asm_simp_tac (simpset() addsimps [comp_sym_iff])));
 by (ALLGOALS (blast_tac (claset() addIs [residuals_preserve_comp, 
 					comp_trans, comp_sym])));
 qed "paving";