Replaced application of subst by simplesubst in proof of app_Var_NF
to avoid problems with program extraction.
--- a/src/HOL/Lambda/WeakNorm.thy Wed Feb 02 18:19:43 2005 +0100
+++ b/src/HOL/Lambda/WeakNorm.thy Wed Feb 02 18:20:31 2005 +0100
@@ -134,7 +134,7 @@
lemma app_Var_NF: "t \<in> NF \<Longrightarrow> \<exists>t'. t \<degree> Var i \<rightarrow>\<^sub>\<beta>\<^sup>* t' \<and> t' \<in> NF"
apply (induct set: NF)
- apply (subst app_last)
+ apply (simplesubst app_last)
apply (rule exI)
apply (rule conjI)
apply (rule rtrancl_refl)