The proper real_alpha
authorCezary Kaliszyk <kaliszyk@in.tum.de>
Fri, 30 Oct 2009 15:22:59 +0100
changeset 242 47de63a883c2
parent 241 60acf3d3a4a0
child 245 55b156ac4a40
The proper real_alpha
LamEx.thy
--- a/LamEx.thy	Fri Oct 30 14:25:37 2009 +0100
+++ b/LamEx.thy	Fri Oct 30 15:22:59 2009 +0100
@@ -78,7 +78,7 @@
   sorry
 
 lemma real_alpha:
-  assumes "t = ([(a,b)]\<bullet>s)" "a\<sharp>s"
+  assumes "t = [(a,b)]\<bullet>s" "a\<sharp>[b].s"
   shows "Lam a t = Lam b s"
 sorry