src/HOL/Nominal/Examples/VC_Condition.thy
changeset 26932 c398a3866082
parent 26262 f5cb9602145f
child 41589 bbd861837ebc
--- a/src/HOL/Nominal/Examples/VC_Condition.thy	Sat May 17 15:31:42 2008 +0200
+++ b/src/HOL/Nominal/Examples/VC_Condition.thy	Sat May 17 21:46:22 2008 +0200
@@ -129,6 +129,7 @@
 lemma false1:
   shows "False"
 proof -
+  fix x
   have "Lam [x].Lam [x].(Var x)\<mapsto>[x,x],(Var x)" 
   and  "\<not>(x\<sharp>Var x)" by (simp_all add: unbind_lambda_lambda1 fresh_atm)
   then have "\<not>(x\<sharp>(bind [x] (Var x)))" by (rule faulty1)
@@ -176,6 +177,7 @@
 lemma false2:
   shows "False"
 proof -
+  fix x
   have "Lam [x].(Var x) \<rightarrow> (Var x)" by (auto intro: strip.intros)
   moreover
   have "x\<sharp>Lam [x].(Var x)" by (simp add: abs_fresh)
@@ -189,6 +191,7 @@
 lemma false3: 
   shows "False"
 proof -
+  fix x
   have "Lam [x].(Var x) \<rightarrow> (Var x)" by (auto intro: strip.intros)
   moreover obtain y::"name" where fc: "y\<sharp>x" by (rule exists_fresh) (rule fin_supp)
   then have "Lam [x].(Var x) = Lam [y].(Var y)"