Nominal/Ex/Term8.thy
changeset 2097 60ce41a11180
parent 2082 0854af516f14
child 2147 e83493622e6f
--- a/Nominal/Ex/Term8.thy	Mon May 10 18:29:45 2010 +0200
+++ b/Nominal/Ex/Term8.thy	Mon May 10 18:32:15 2010 +0200
@@ -7,7 +7,7 @@
 atom_decl name
 
 (* this should work but gives an error at the moment:
-   seems like in the symmetry proof
+   in alpha_bn_rsp proof.
 *)
 
 nominal_datatype foo =
@@ -15,7 +15,7 @@
 | Foo1 b::"bar" f::"foo" bind_set "bv b" in f
 and bar =
   Bar0 "name"
-| Bar1 "name" s::"name" b::"bar" bind s in b
+| Bar1 "name" s::"name" b::"bar" bind_set s in b
 binder
   bv
 where