src/HOL/HOLCF/IOA/meta_theory/Automata.thy
changeset 44066 d74182c93f04
parent 42793 88bee9f6eec7
child 45606 b1e1508643b1
equal deleted inserted replaced
44065:eb64ffccfc75 44066:d74182c93f04
   607       (fst(snd(snd(s))),a,fst(snd(snd(t)))):trans_of(C)                       
   607       (fst(snd(snd(s))),a,fst(snd(snd(t)))):trans_of(C)                       
   608     else fst(snd(snd(t)))=fst(snd(snd(s)))) &                                 
   608     else fst(snd(snd(t)))=fst(snd(snd(s)))) &                                 
   609    (if a:actions(asig_of(D)) then                                             
   609    (if a:actions(asig_of(D)) then                                             
   610       (snd(snd(snd(s))),a,snd(snd(snd(t)))):trans_of(D)                       
   610       (snd(snd(snd(s))),a,snd(snd(snd(t)))):trans_of(D)                       
   611     else snd(snd(snd(t)))=snd(snd(snd(s)))))"
   611     else snd(snd(snd(t)))=snd(snd(snd(s)))))"
   612   apply (simp (no_asm) add: par_def actions_asig_comp Pair_fst_snd_eq Let_def ioa_projections)
   612   apply (simp (no_asm) add: par_def actions_asig_comp prod_eq_iff Let_def ioa_projections)
   613   done
   613   done
   614 
   614 
   615 
   615 
   616 subsection "proof obligation generator for IOA requirements"
   616 subsection "proof obligation generator for IOA requirements"
   617 
   617