src/HOL/UNITY/Comp/Counter.thy
changeset 16417 9bc16273c2d4
parent 16184 80617b8d33c5
child 18556 dc39832e9280
equal deleted inserted replaced
16416:6061ae1f90f2 16417:9bc16273c2d4
     9    Spriner LNCS 1586 (1999), pages 1215-1227.
     9    Spriner LNCS 1586 (1999), pages 1215-1227.
    10 *)
    10 *)
    11 
    11 
    12 header{*A Family of Similar Counters: Original Version*}
    12 header{*A Family of Similar Counters: Original Version*}
    13 
    13 
    14 theory Counter = UNITY_Main:
    14 theory Counter imports UNITY_Main begin
    15 
    15 
    16 (* Variables are names *)
    16 (* Variables are names *)
    17 datatype name = C | c nat
    17 datatype name = C | c nat
    18 types state = "name=>int"
    18 types state = "name=>int"
    19 
    19