--- a/src/FOL/IFOL.thy Mon Feb 08 21:26:52 2010 +0100
+++ b/src/FOL/IFOL.thy Mon Feb 08 21:28:27 2010 +0100
@@ -772,7 +772,7 @@
translations
"_Let(_binds(b, bs), e)" == "_Let(b, _Let(bs, e))"
- "let x = a in e" == "Let(a, %x. e)"
+ "let x = a in e" == "CONST Let(a, %x. e)"
lemma LetI: