src/HOL/TLA/Action.thy
changeset 55382 9218fa411c15
parent 54742 7a86358a3c0b
child 56256 1e01c159e7d9
equal deleted inserted replaced
55381:ca31f042414f 55382:9218fa411c15
    13 (** abstract syntax **)
    13 (** abstract syntax **)
    14 
    14 
    15 type_synonym 'a trfun = "(state * state) => 'a"
    15 type_synonym 'a trfun = "(state * state) => 'a"
    16 type_synonym action   = "bool trfun"
    16 type_synonym action   = "bool trfun"
    17 
    17 
    18 arities prod :: (world, world) world
    18 instance prod :: (world, world) world ..
    19 
    19 
    20 consts
    20 consts
    21   (** abstract syntax **)
    21   (** abstract syntax **)
    22   before        :: "'a stfun => 'a trfun"
    22   before        :: "'a stfun => 'a trfun"
    23   after         :: "'a stfun => 'a trfun"
    23   after         :: "'a stfun => 'a trfun"