src/HOL/UNITY/Simple/Common.thy
changeset 18556 dc39832e9280
parent 16417 9bc16273c2d4
child 21026 3b2821e0d541
equal deleted inserted replaced
18555:5f216b70215f 18556:dc39832e9280
     8 The state is identified with the one variable in existence.
     8 The state is identified with the one variable in existence.
     9 
     9 
    10 From Misra, "A Logic for Concurrent Programming" (1994), sections 5.1 and 13.1.
    10 From Misra, "A Logic for Concurrent Programming" (1994), sections 5.1 and 13.1.
    11 *)
    11 *)
    12 
    12 
    13 theory Common imports UNITY_Main begin
    13 theory Common imports "../UNITY_Main" begin
    14 
    14 
    15 consts
    15 consts
    16   ftime :: "nat=>nat"
    16   ftime :: "nat=>nat"
    17   gtime :: "nat=>nat"
    17   gtime :: "nat=>nat"
    18 
    18