Nominal/Ex/LetSimple2.thy
changeset 2950 0911cb7bf696
parent 2943 09834ba7ce59
child 2960 248546bfeb16
--- a/Nominal/Ex/LetSimple2.thy	Tue Jul 05 18:01:54 2011 +0200
+++ b/Nominal/Ex/LetSimple2.thy	Tue Jul 05 18:42:34 2011 +0200
@@ -7,7 +7,7 @@
 nominal_datatype trm =
   Var "name"
 | App "trm" "trm"
-| Let as::"assn" t::"trm"   bind "bn as" in t
+| Let as::"assn" t::"trm"   binds "bn as" in t
 and assn =
   Assn "name" "trm"
 binder