Nominal/Ex/LetRecB.thy
changeset 2950 0911cb7bf696
parent 2922 a27215ab674e
--- a/Nominal/Ex/LetRecB.thy	Tue Jul 05 18:01:54 2011 +0200
+++ b/Nominal/Ex/LetRecB.thy	Tue Jul 05 18:42:34 2011 +0200
@@ -8,8 +8,8 @@
  trm =
   Var "name"
 | App "trm" "trm"
-| Lam x::"name" t::"trm"     bind x in t
-| Let_Rec bp::"bp" t::"trm"  bind "bn bp" in bp t
+| Lam x::"name" t::"trm"     binds x in t
+| Let_Rec bp::"bp" t::"trm"  binds "bn bp" in bp t
 and bp =
   Bp "name" "trm"
 binder