author | paulson |
Tue, 10 May 2005 10:25:21 +0200 | |
changeset 15948 | d97c12a4f31b |
parent 15947 | 393cfc718433 |
child 15949 | fd02dd265b78 |
--- a/src/HOL/Lambda/WeakNorm.thy Tue May 10 06:59:32 2005 +0200 +++ b/src/HOL/Lambda/WeakNorm.thy Tue May 10 10:25:21 2005 +0200 @@ -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) --{*Using @{text subst} makes extraction fail*} apply (rule exI) apply (rule conjI) apply (rule rtrancl_refl)