src/HOL/Proofs/Lambda/NormalForm.thy
changeset 67443 3abf6a722518
parent 61986 2461779da2b8
child 69597 ff784d5a5bfb
--- a/src/HOL/Proofs/Lambda/NormalForm.thy	Tue Jan 16 09:12:16 2018 +0100
+++ b/src/HOL/Proofs/Lambda/NormalForm.thy	Tue Jan 16 09:30:00 2018 +0100
@@ -146,7 +146,7 @@
 
 lemma app_Var_NF: "NF t \<Longrightarrow> \<exists>t'. t \<degree> Var i \<rightarrow>\<^sub>\<beta>\<^sup>* t' \<and> NF t'"
   apply (induct set: NF)
-  apply (simplesubst app_last)  \<comment>\<open>Using \<open>subst\<close> makes extraction fail\<close>
+  apply (simplesubst app_last)  \<comment> \<open>Using \<open>subst\<close> makes extraction fail\<close>
   apply (rule exI)
   apply (rule conjI)
   apply (rule rtranclp.rtrancl_refl)