src/HOL/UNITY/Comp/Alloc.thy
changeset 30510 4120fc59dd85
parent 25995 21b51f748daf
child 30528 7173bf123335
equal deleted inserted replaced
30509:e19d5b459a61 30510:4120fc59dd85
   319       @{thm client_map_def}, @{thm non_dummy_def}, @{thm funPair_def},
   319       @{thm client_map_def}, @{thm non_dummy_def}, @{thm funPair_def},
   320       @{thm o_apply}, @{thm Let_def}])
   320       @{thm o_apply}, @{thm Let_def}])
   321 *}
   321 *}
   322 
   322 
   323 method_setup record_auto = {*
   323 method_setup record_auto = {*
   324   Method.ctxt_args (fn ctxt => Method.SIMPLE_METHOD (record_auto_tac (local_clasimpset_of ctxt)))
   324   Method.ctxt_args (fn ctxt => SIMPLE_METHOD (record_auto_tac (local_clasimpset_of ctxt)))
   325 *} ""
   325 *} ""
   326 
   326 
   327 lemma inj_sysOfAlloc [iff]: "inj sysOfAlloc"
   327 lemma inj_sysOfAlloc [iff]: "inj sysOfAlloc"
   328   apply (unfold sysOfAlloc_def Let_def)
   328   apply (unfold sysOfAlloc_def Let_def)
   329   apply (rule inj_onI)
   329   apply (rule inj_onI)
   712         (@{simpset} addsimps [@{thm o_def}, @{thm non_dummy_def}, @{thm guarantees_Int_right}]) 1]
   712         (@{simpset} addsimps [@{thm o_def}, @{thm non_dummy_def}, @{thm guarantees_Int_right}]) 1]
   713 *}
   713 *}
   714 
   714 
   715 method_setup rename_client_map = {*
   715 method_setup rename_client_map = {*
   716   Method.ctxt_args (fn ctxt =>
   716   Method.ctxt_args (fn ctxt =>
   717     Method.SIMPLE_METHOD (rename_client_map_tac (local_simpset_of ctxt)))
   717     SIMPLE_METHOD (rename_client_map_tac (local_simpset_of ctxt)))
   718 *} ""
   718 *} ""
   719 
   719 
   720 text{*Lifting @{text Client_Increasing} to @{term systemState}*}
   720 text{*Lifting @{text Client_Increasing} to @{term systemState}*}
   721 lemma rename_Client_Increasing: "i : I
   721 lemma rename_Client_Increasing: "i : I
   722       ==> rename sysOfClient (plam x: I. rename client_map Client) :
   722       ==> rename sysOfClient (plam x: I. rename client_map Client) :