diff -r e1fce873b814 -r d797baa3d57c src/FOL/IFOL.thy --- a/src/FOL/IFOL.thy Fri Dec 17 17:08:56 2010 +0100 +++ b/src/FOL/IFOL.thy Fri Dec 17 17:43:54 2010 +0100 @@ -754,7 +754,7 @@ subsection {* ``Let'' declarations *} -nonterminals letbinds letbind +nonterminal letbinds and letbind definition Let :: "['a::{}, 'a => 'b] => ('b::{})" where "Let(s, f) == f(s)"