src/HOL/TLA/Action.thy
changeset 37678 0040bafffdef
parent 35354 2e8dc3c64430
child 42018 878f33040280
equal deleted inserted replaced
37677:c5a8b612e571 37678:0040bafffdef
    14 
    14 
    15 types
    15 types
    16   'a trfun = "(state * state) => 'a"
    16   'a trfun = "(state * state) => 'a"
    17   action   = "bool trfun"
    17   action   = "bool trfun"
    18 
    18 
    19 arities
    19 arities prod :: (world, world) world
    20   "*" :: (world, world) world
       
    21 
    20 
    22 consts
    21 consts
    23   (** abstract syntax **)
    22   (** abstract syntax **)
    24   before        :: "'a stfun => 'a trfun"
    23   before        :: "'a stfun => 'a trfun"
    25   after         :: "'a stfun => 'a trfun"
    24   after         :: "'a stfun => 'a trfun"