src/HOLCF/IOA/meta_theory/TLS.thy
changeset 36452 d37c6eed8117
parent 35215 a03462cbf86f
child 37598 893dcabf0c04
equal deleted inserted replaced
36451:ddc965e172c4 36452:d37c6eed8117
     6 
     6 
     7 theory TLS
     7 theory TLS
     8 imports IOA TL
     8 imports IOA TL
     9 begin
     9 begin
    10 
    10 
    11 defaultsort type
    11 default_sort type
    12 
    12 
    13 types
    13 types
    14   ('a, 's) ioa_temp  = "('a option,'s)transition temporal"
    14   ('a, 's) ioa_temp  = "('a option,'s)transition temporal"
    15   ('a, 's) step_pred = "('a option,'s)transition predicate"
    15   ('a, 's) step_pred = "('a option,'s)transition predicate"
    16   's state_pred      = "'s predicate"
    16   's state_pred      = "'s predicate"