Nominal/Parser.thy
changeset 1434 d2d8020cd20a
parent 1433 7a9217a7f681
child 1436 04dad9b0136d
--- a/Nominal/Parser.thy	Thu Mar 11 20:49:31 2010 +0100
+++ b/Nominal/Parser.thy	Fri Mar 12 12:42:35 2010 +0100
@@ -510,7 +510,7 @@
   fun prep_bn env bn_str =
     case (Syntax.read_term lthy bn_str) of
        Free (x, _) => (NONE, env_lookup env x)
-     | Const (a, T) $ Free (x, _) => (SOME (Const (a, T), false), env_lookup env x)
+     | Const (a, T) $ Free (x, _) => (SOME (Const (a, T), true), env_lookup env x)
      | _ => error (bn_str ^ " not allowed as binding specification.");  
  
   fun prep_typ env (i, opt_name) =