src/HOL/HOLCF/IOA/meta_theory/TLS.thy
changeset 62003 ba465fcd0267
parent 62002 f1599e98c4d0
child 62005 68db98c2cd97
equal deleted inserted replaced
62002:f1599e98c4d0 62003:ba465fcd0267
   161 
   161 
   162 (* uses the fact that in executions states overlap, which is lost in 
   162 (* uses the fact that in executions states overlap, which is lost in 
   163    after the translation via ex2seq !! *)
   163    after the translation via ex2seq !! *)
   164 
   164 
   165 lemma TL_TLS: 
   165 lemma TL_TLS: 
   166  "[| ! s a t. (P s) & s-a--A-> t --> (Q t) |] 
   166  "[| ! s a t. (P s) & s \<midarrow>a\<midarrow>A\<rightarrow> t --> (Q t) |] 
   167    ==> ex \<TTurnstile> (Init (%(s,a,t). P s) \<^bold>\<and> Init (%(s,a,t). s -a--A-> t)  
   167    ==> ex \<TTurnstile> (Init (%(s,a,t). P s) \<^bold>\<and> Init (%(s,a,t). s \<midarrow>a\<midarrow>A\<rightarrow> t)  
   168               \<^bold>\<longrightarrow> (Next (Init (%(s,a,t).Q s))))"
   168               \<^bold>\<longrightarrow> (Next (Init (%(s,a,t).Q s))))"
   169 apply (unfold Init_def Next_def temp_sat_def satisfies_def IMPLIES_def AND_def)
   169 apply (unfold Init_def Next_def temp_sat_def satisfies_def IMPLIES_def AND_def)
   170 
   170 
   171 apply clarify
   171 apply clarify
   172 apply (simp split add: split_if)
   172 apply (simp split add: split_if)