changeset 52143 | 36ffe23b25f8 |
parent 50105 | 65d5b18e1626 |
child 54295 | 45a5523d4a63 |
--- a/src/HOL/Hilbert_Choice.thy Sat May 25 15:00:53 2013 +0200 +++ b/src/HOL/Hilbert_Choice.thy Sat May 25 15:37:53 2013 +0200 @@ -25,7 +25,7 @@ "SOME x. P" == "CONST Eps (%x. P)" print_translation {* - [(@{const_syntax Eps}, fn [Abs abs] => + [(@{const_syntax Eps}, fn _ => fn [Abs abs] => let val (x, t) = Syntax_Trans.atomic_abs_tr' abs in Syntax.const @{syntax_const "_Eps"} $ x $ t end)] *} -- {* to avoid eta-contraction of body *}