diff -r a1a251b297dd -r 1b3780be6cc2 src/HOL/Lambda/ListBeta.thy --- a/src/HOL/Lambda/ListBeta.thy Thu Feb 16 21:11:58 2006 +0100 +++ b/src/HOL/Lambda/ListBeta.thy Thu Feb 16 21:12:00 2006 +0100 @@ -12,10 +12,9 @@ Lifting beta-reduction to lists of terms, reducing exactly one element. *} -syntax - "_list_beta" :: "dB => dB => bool" (infixl "=>" 50) -translations - "rs => ss" == "(rs, ss) : step1 beta" +abbreviation (output) + list_beta :: "dB list => dB list => bool" (infixl "=>" 50) + "(rs => ss) = ((rs, ss) : step1 beta)" lemma head_Var_reduction: "Var n \\ rs -> v \ \ss. rs => ss \ v = Var n \\ ss"