src/HOL/Nominal/Examples/Lam_Funs.thy
changeset 22832 6a16085eaaa1
parent 22829 f1db55c7534d
child 25751 a4e69ce247e0
--- a/src/HOL/Nominal/Examples/Lam_Funs.thy	Thu May 03 17:54:36 2007 +0200
+++ b/src/HOL/Nominal/Examples/Lam_Funs.thy	Thu May 03 19:00:28 2007 +0200
@@ -67,9 +67,6 @@
 
 lemma subst_eqvt[eqvt]:
   fixes pi:: "name prm"
-  and   t1:: "lam"
-  and   t2:: "lam"
-  and   a :: "name"
   shows "pi\<bullet>(t1[b::=t2]) = (pi\<bullet>t1)[(pi\<bullet>b)::=(pi\<bullet>t2)]"
 apply(nominal_induct t1 avoiding: b t2 rule: lam.induct)
 apply(auto simp add: perm_bij fresh_prod fresh_atm fresh_bij)
@@ -95,8 +92,6 @@
 
 lemma lookup_eqvt[eqvt]:
   fixes pi::"name prm"
-  and   \<theta>::"(name\<times>lam) list"
-  and   x::"name"
   shows "pi\<bullet>(lookup \<theta> x) = lookup (pi\<bullet>\<theta>) (pi\<bullet>x)"
 by (induct \<theta>) (auto simp add: perm_bij)