src/FOL/IFOL.thy
changeset 35054 a5db9779b026
parent 33369 470a7b233ee5
child 35409 5c5bb83f2bae
child 35416 d8d7d1b785af
--- 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: