src/HOL/Lambda/WeakNorm.thy
changeset 15948 d97c12a4f31b
parent 15944 9b00875e21f7
child 16417 9bc16273c2d4
equal deleted inserted replaced
15947:393cfc718433 15948:d97c12a4f31b
   132   apply (rules intro: NF.Abs)
   132   apply (rules intro: NF.Abs)
   133   done
   133   done
   134 
   134 
   135 lemma app_Var_NF: "t \<in> NF \<Longrightarrow> \<exists>t'. t \<degree> Var i \<rightarrow>\<^sub>\<beta>\<^sup>* t' \<and> t' \<in> NF"
   135 lemma app_Var_NF: "t \<in> NF \<Longrightarrow> \<exists>t'. t \<degree> Var i \<rightarrow>\<^sub>\<beta>\<^sup>* t' \<and> t' \<in> NF"
   136   apply (induct set: NF)
   136   apply (induct set: NF)
   137   apply (subst app_last)
   137   apply (simplesubst app_last)  --{*Using @{text subst} makes extraction fail*}
   138   apply (rule exI)
   138   apply (rule exI)
   139   apply (rule conjI)
   139   apply (rule conjI)
   140   apply (rule rtrancl_refl)
   140   apply (rule rtrancl_refl)
   141   apply (rule NF.App)
   141   apply (rule NF.App)
   142   apply (drule listall_conj1)
   142   apply (drule listall_conj1)