src/HOL/TLA/TLA.thy
changeset 35068 544867142ea4
parent 30528 7173bf123335
child 35108 e384e27c229f
equal deleted inserted replaced
35067:af4c18c30593 35068:544867142ea4
    35 
    35 
    36   "_EEx"     :: "[idts, lift] => lift"                ("(3EEX _./ _)" [0,10] 10)
    36   "_EEx"     :: "[idts, lift] => lift"                ("(3EEX _./ _)" [0,10] 10)
    37   "_AAll"    :: "[idts, lift] => lift"                ("(3AALL _./ _)" [0,10] 10)
    37   "_AAll"    :: "[idts, lift] => lift"                ("(3AALL _./ _)" [0,10] 10)
    38 
    38 
    39 translations
    39 translations
    40   "_Box"      ==   "Box"
    40   "_Box"      ==   "CONST Box"
    41   "_Dmd"      ==   "Dmd"
    41   "_Dmd"      ==   "CONST Dmd"
    42   "_leadsto"  ==   "leadsto"
    42   "_leadsto"  ==   "CONST leadsto"
    43   "_stable"   ==   "Stable"
    43   "_stable"   ==   "CONST Stable"
    44   "_WF"       ==   "WF"
    44   "_WF"       ==   "CONST WF"
    45   "_SF"       ==   "SF"
    45   "_SF"       ==   "CONST SF"
    46   "_EEx v A"  ==   "Eex v. A"
    46   "_EEx v A"  ==   "Eex v. A"
    47   "_AAll v A" ==   "Aall v. A"
    47   "_AAll v A" ==   "Aall v. A"
    48 
    48 
    49   "sigma |= []F"         <= "_Box F sigma"
    49   "sigma |= []F"         <= "_Box F sigma"
    50   "sigma |= <>F"         <= "_Dmd F sigma"
    50   "sigma |= <>F"         <= "_Dmd F sigma"