src/ZF/UNITY/State.thy
changeset 58871 c399ae4b836f
parent 46823 57bf0cecb366
child 60770 240563fbf41d
equal deleted inserted replaced
58870:e2c0d8ef29cb 58871:c399ae4b836f
     6  - variables are typed.
     6  - variables are typed.
     7  - the state space is uniform, common to all defined programs.
     7  - the state space is uniform, common to all defined programs.
     8  - variables can be quantified over.
     8  - variables can be quantified over.
     9 *)
     9 *)
    10 
    10 
    11 header{*UNITY Program States*}
    11 section{*UNITY Program States*}
    12 
    12 
    13 theory State imports Main begin
    13 theory State imports Main begin
    14 
    14 
    15 consts var :: i
    15 consts var :: i
    16 datatype var = Var("i \<in> list(nat)")
    16 datatype var = Var("i \<in> list(nat)")