src/HOLCF/IOA/meta_theory/ShortExecutions.thy
author wenzelm
Sat, 03 Nov 2001 01:39:17 +0100
changeset 12028 52aa183c15bb
parent 10835 f4745d77e620
child 12218 6597093b77e7
permissions -rw-r--r--
replaced Undef by UU;

(*  Title:      HOLCF/IOA/meta_theory/ShortExecutions.thy
    ID:         $Id$
    Author:     Olaf M"uller
    Copyright   1997  TU Muenchen

Some properties about (Cut ex), defined as follows:

For every execution ex there is another shorter execution (Cut ex) 
that has the same trace as ex, but its schedule ends with an external action.

*) 


ShortExecutions = Traces + 

consts 

(*  LastActExtex      ::"('a,'s)ioa => ('a,'s) pairs  => bool"*)
  LastActExtsch     ::"('a,'s)ioa => 'a Seq         => bool"

  Cut               ::"('a => bool) => 'a Seq    => 'a Seq"
 
  oraclebuild       ::"('a => bool) => 'a Seq -> 'a Seq -> 'a Seq"

defs

LastActExtsch_def
  "LastActExtsch A sch == (Cut (%x. x: ext A) sch = sch)"

(* LastActExtex_def
  "LastActExtex A ex == LastActExtsch A (filter_act$ex)" *)

Cut_def
  "Cut P s == oraclebuild P$s$(Filter P$s)"

oraclebuild_def
  "oraclebuild P == (fix$(LAM h s t. case t of 
       nil => nil
    | x##xs => 
      (case x of 
        UU => UU
      | Def y => (Takewhile (%x.~P x)$s)
                  @@ (y>>(h$(TL$(Dropwhile (%x.~ P x)$s))$xs))
      )
    ))"




rules

Cut_prefixcl_Finite
  "Finite s ==> (? y. s = Cut P s @@ y)"

LastActExtsmall1
  "LastActExtsch A sch ==> LastActExtsch A (TL$(Dropwhile P$sch))"

LastActExtsmall2
  "[| Finite sch1; LastActExtsch A (sch1 @@ sch2) |] ==> LastActExtsch A sch2"

end