commented out parts which have been inactive (unintentionally) for a long time;
authorwenzelm
Tue, 07 Nov 2006 14:30:00 +0100
changeset 21220 63a7a74a9489
parent 21219 e1063a0e6dfd
child 21221 ef30d1e6f03a
commented out parts which have been inactive (unintentionally) for a long time;
src/HOL/UNITY/Comp/Alloc.ML
--- a/src/HOL/UNITY/Comp/Alloc.ML	Tue Nov 07 14:29:58 2006 +0100
+++ b/src/HOL/UNITY/Comp/Alloc.ML	Tue Nov 07 14:30:00 2006 +0100
@@ -348,7 +348,7 @@
 by (dres_inst_tac [("w1", "ask")] (impOfSubs subset_preserves_o) 2);
 by (auto_tac (claset(), simpset() addsimps [o_def, split_def]));  
 qed "OK_lift_rename_Client";
-Addsimps [OK_lift_rename_Client]; (*needed in rename_client_map_tac*
+Addsimps [OK_lift_rename_Client]; (*needed in rename_client_map_tac*)
 
 (*The proofs of rename_Client_Increasing, rename_Client_Bounded and
   rename_Client_Progress are similar.  All require copying out the original
@@ -385,6 +385,8 @@
         (simpset() addsimps [o_def, non_dummy_def, guarantees_Int_right]) 1];
 
 						     
+(* FIXME no longer works -- had been commented out unintentially for a long time
+
 (*Lifting Client_Increasing to systemState*)
 Goal "i : I \
 \     ==> rename sysOfClient (plam x: I. rename client_map Client) : \
@@ -740,3 +742,4 @@
 by (asm_full_simp_tac (simpset() addsimps [bij_is_inj, inv_f_f]) 1); 
 by (asm_full_simp_tac (simpset() addsimps [bij_is_surj, surj_f_inv_f]) 1); 
 qed "bij_fst_inv_inv_eq";
+*)