src/HOL/TLA/Stfun.thy
changeset 35354 2e8dc3c64430
parent 35318 e1b61c5fd494
child 42018 878f33040280
equal deleted inserted replaced
35353:1391f82da5a4 35354:2e8dc3c64430
    33      "meta predicate" basevars, which is defined here.
    33      "meta predicate" basevars, which is defined here.
    34   *)
    34   *)
    35   stvars    :: "'a stfun => bool"
    35   stvars    :: "'a stfun => bool"
    36 
    36 
    37 syntax
    37 syntax
    38   "PRED"    :: "lift => 'a"                          ("PRED _")
    38   "_PRED"   :: "lift => 'a"                          ("PRED _")
    39   "_stvars" :: "lift => bool"                        ("basevars _")
    39   "_stvars" :: "lift => bool"                        ("basevars _")
    40 
    40 
    41 translations
    41 translations
    42   "PRED P"   =>  "(P::state => _)"
    42   "PRED P"   =>  "(P::state => _)"
    43   "_stvars"  ==  "CONST stvars"
    43   "_stvars"  ==  "CONST stvars"