src/HOL/Lambda/ParRed.thy
changeset 8624 69619f870939
parent 5146 1ea751ae62b2
child 9811 39ffdb8cab03
equal deleted inserted replaced
8623:5668aaf41c36 8624:69619f870939
     4     Copyright   1995 TU Muenchen
     4     Copyright   1995 TU Muenchen
     5 
     5 
     6 Parallel reduction and a complete developments function "cd".
     6 Parallel reduction and a complete developments function "cd".
     7 *)
     7 *)
     8 
     8 
     9 ParRed = Lambda + Commutation + Recdef +
     9 ParRed = Lambda + Commutation +
    10 
    10 
    11 consts  par_beta :: "(dB * dB) set"
    11 consts  par_beta :: "(dB * dB) set"
    12 
    12 
    13 syntax  "=>" :: [dB,dB] => bool (infixl 50)
    13 syntax  "=>" :: [dB,dB] => bool (infixl 50)
    14 
    14