Nominal/Ex/CoreHaskell2.thy
changeset 2950 0911cb7bf696
parent 2617 e44551d067e6
--- a/Nominal/Ex/CoreHaskell2.thy	Tue Jul 05 18:01:54 2011 +0200
+++ b/Nominal/Ex/CoreHaskell2.thy	Tue Jul 05 18:42:34 2011 +0200
@@ -20,7 +20,7 @@
        Tvar tvar
      | Tcon string
      | Tapp Ty Ty
-     | Tforall pb::PBind ty::Ty   bind "bind_pb pb" in ty
+     | Tforall pb::PBind ty::Ty   binds "bind_pb pb" in ty
 and PBind =
   Pbind tvar Kind
 binder
@@ -37,7 +37,7 @@
      | Dcon string
      | App Exp Exp
      | Appt Exp Ty
-     | Lam b::Bind e::Exp bind "bind_b b" in e
+     | Lam b::Bind e::Exp binds "bind_b b" in e
 binder
   bind_b
 where