src/HOL/Hoare_Parallel/RG_Com.thy
author immler
Wed, 12 Nov 2014 17:36:36 +0100
changeset 58984 ae0c56c485ae
parent 58884 be4d203d35b3
child 59189 ad8e0a789af6
permissions -rw-r--r--
added lemmas: convert between powr and log in comparisons, pull log out of addition/subtraction

chapter {* The Rely-Guarantee Method *}

section {* Abstract Syntax *}

theory RG_Com imports Main begin

text {* Semantics of assertions and boolean expressions (bexp) as sets
of states.  Syntax of commands @{text com} and parallel commands
@{text par_com}. *}

type_synonym 'a bexp = "'a set"

datatype 'a com = 
    Basic "'a \<Rightarrow>'a"
  | Seq "'a com" "'a com"
  | Cond "'a bexp" "'a com" "'a com"         
  | While "'a bexp" "'a com"       
  | Await "'a bexp" "'a com"                 

type_synonym 'a par_com = "'a com option list"

end