src/HOL/HOLCF/IOA/meta_theory/TLS.thy
changeset 41476 0fa9629aa399
parent 40945 b8703f63bfb2
child 42151 4da4fc77664b
equal deleted inserted replaced
41468:0e4f6cf20cdf 41476:0fa9629aa399
     8 imports IOA TL
     8 imports IOA TL
     9 begin
     9 begin
    10 
    10 
    11 default_sort type
    11 default_sort type
    12 
    12 
    13 types
    13 type_synonym
    14   ('a, 's) ioa_temp  = "('a option,'s)transition temporal"
    14   ('a, 's) ioa_temp  = "('a option,'s)transition temporal"
       
    15 
       
    16 type_synonym
    15   ('a, 's) step_pred = "('a option,'s)transition predicate"
    17   ('a, 's) step_pred = "('a option,'s)transition predicate"
       
    18 
       
    19 type_synonym
    16   's state_pred      = "'s predicate"
    20   's state_pred      = "'s predicate"
    17 
    21 
    18 consts
    22 consts
    19 
    23 
    20 option_lift :: "('a => 'b) => 'b => ('a option => 'b)"
    24 option_lift :: "('a => 'b) => 'b => ('a option => 'b)"