Nominal/Ex/SingleLet.thy
changeset 2213 231a20534950
parent 2200 31f1ec832d39
child 2284 7b83e1c8ba2e
child 2312 ad03df7e8056
child 2326 b51532dd5689
--- a/Nominal/Ex/SingleLet.thy	Sun Jun 06 13:16:27 2010 +0200
+++ b/Nominal/Ex/SingleLet.thy	Mon Jun 07 11:33:00 2010 +0200
@@ -8,7 +8,8 @@
   Var "name"
 | App "trm" "trm"
 | Lam x::"name" t::"trm"  bind_set x in t
-| Let a::"assg" t::"trm"  bind_set "bn a" in t
+| Let a::"assg" t1::"trm" t2::"trm" bind_set "bn a" in t1 t2
+ 
 and assg =
   As "name" "trm"
 binder