src/HOLCF/IOA/meta_theory/TL.thy
changeset 12338 de0f4a63baa5
parent 12218 6597093b77e7
child 14981 e73f8140af78
equal deleted inserted replaced
12337:7c6a970f0808 12338:de0f4a63baa5
     6 A General Temporal Logic.
     6 A General Temporal Logic.
     7 *)   
     7 *)   
     8 	       
     8 	       
     9 TL = Pred + Sequence +  
     9 TL = Pred + Sequence +  
    10 
    10 
    11 default term
    11 default type
    12 
    12 
    13 types
    13 types
    14 
    14 
    15 'a temporal      = 'a Seq predicate
    15 'a temporal      = 'a Seq predicate
    16 
    16