src/HOL/UNITY/Comp/Counterc.thy
changeset 12338 de0f4a63baa5
parent 11868 56db9f3a6b3e
child 13792 d1811693899c
equal deleted inserted replaced
12337:7c6a970f0808 12338:de0f4a63baa5
    11    Spriner LNCS 1586 (1999), pages 1215-1227.
    11    Spriner LNCS 1586 (1999), pages 1215-1227.
    12 *)
    12 *)
    13 
    13 
    14 Counterc =  Comp +
    14 Counterc =  Comp +
    15 types state
    15 types state
    16 arities state :: term
    16 arities state :: type
    17 
    17 
    18 consts
    18 consts
    19   C :: "state=>int"
    19   C :: "state=>int"
    20   c :: "state=>nat=>int"
    20   c :: "state=>nat=>int"
    21 
    21