turing_basic.thy
changeset 41 6d89ed67ba27
parent 0 aa8656a8dbef
child 50 816e84ca16d6
equal deleted inserted replaced
40:a37a21f7ccf4 41:6d89ed67ba27
   619 text {*
   619 text {*
   620   The following lemma tries to derive the Hoare logic rule for sequentially combined TMs.
   620   The following lemma tries to derive the Hoare logic rule for sequentially combined TMs.
   621   It deals with the situtation when both @{text "A"} and @{text "B"} are terminated.
   621   It deals with the situtation when both @{text "A"} and @{text "B"} are terminated.
   622 *}
   622 *}
   623 
   623 
       
   624 thm t_merge_pre_halt_same
       
   625 
   624 lemma t_merge_halt: 
   626 lemma t_merge_halt: 
   625   assumes aimpb: "Q1 \<turnstile>-> P2"
   627   assumes aimpb: "Q1 \<turnstile>-> P2"
   626   shows "P1 \<turnstile>->  \<lambda> tp. (\<exists> stp tp'. steps (Suc 0, tp) (A |+| B)  stp = (0, tp') \<and> Q2 tp')"
   628   shows "P1 \<turnstile>->  \<lambda> tp. (\<exists> stp tp'. steps (Suc 0, tp) (A |+| B)  stp = (0, tp') \<and> Q2 tp')"
   627 proof(simp add: t_imply_def, auto)
   629 proof(simp add: t_imply_def, auto)
   628   fix a b
   630   fix a b