diff -r a1a251b297dd -r 1b3780be6cc2 src/HOL/Lambda/Lambda.thy --- a/src/HOL/Lambda/Lambda.thy Thu Feb 16 21:11:58 2006 +0100 +++ b/src/HOL/Lambda/Lambda.thy Thu Feb 16 21:12:00 2006 +0100 @@ -56,15 +56,15 @@ consts beta :: "(dB \ dB) set" -syntax - "_beta" :: "[dB, dB] => bool" (infixl "->" 50) - "_beta_rtrancl" :: "[dB, dB] => bool" (infixl "->>" 50) +abbreviation (output) + beta_red :: "[dB, dB] => bool" (infixl "->" 50) + "(s -> t) = ((s, t) \ beta)" + beta_reds :: "[dB, dB] => bool" (infixl "->>" 50) + "(s ->> t) = ((s, t) \ beta^*)" + syntax (latex) - "_beta" :: "[dB, dB] => bool" (infixl "\\<^sub>\" 50) - "_beta_rtrancl" :: "[dB, dB] => bool" (infixl "\\<^sub>\\<^sup>*" 50) -translations - "s \\<^sub>\ t" == "(s, t) \ beta" - "s \\<^sub>\\<^sup>* t" == "(s, t) \ beta^*" + beta_red :: "[dB, dB] => bool" (infixl "\\<^sub>\" 50) + beta_reds :: "[dB, dB] => bool" (infixl "\\<^sub>\\<^sup>*" 50) inductive beta intros