Nominal/Ex/SingleLet.thy
changeset 2284 7b83e1c8ba2e
parent 2213 231a20534950
child 2318 49cc1af89de9
child 2327 bcb037806e16
--- a/Nominal/Ex/SingleLet.thy	Sun Jun 20 02:37:44 2010 +0100
+++ b/Nominal/Ex/SingleLet.thy	Sun Jun 20 02:37:58 2010 +0100
@@ -8,7 +8,7 @@
   Var "name"
 | App "trm" "trm"
 | Lam x::"name" t::"trm"  bind_set x in t
-| Let a::"assg" t1::"trm" t2::"trm" bind_set "bn a" in t1 t2
+| Let a::"assg" t::"trm" bind_set "bn a" in t
  
 and assg =
   As "name" "trm"