src/HOL/Proofs/Lambda/StrongNorm.thy
changeset 69597 ff784d5a5bfb
parent 61986 2461779da2b8
child 76987 4c275405faae
--- a/src/HOL/Proofs/Lambda/StrongNorm.thy	Sat Jan 05 17:00:43 2019 +0100
+++ b/src/HOL/Proofs/Lambda/StrongNorm.thy	Sat Jan 05 17:24:33 2019 +0100
@@ -36,7 +36,7 @@
 
 lemma subst_Var_IT: "IT r \<Longrightarrow> IT (r[Var i/j])"
   apply (induct arbitrary: i j set: IT)
-    txt \<open>Case @{term Var}:\<close>
+    txt \<open>Case \<^term>\<open>Var\<close>:\<close>
     apply (simp (no_asm) add: subst_Var)
     apply
     ((rule conjI impI)+,
@@ -47,12 +47,12 @@
       rule listsp.Cons,
       fast,
       assumption)+
-   txt \<open>Case @{term Lambda}:\<close>
+   txt \<open>Case \<^term>\<open>Lambda\<close>:\<close>
    apply atomize
    apply simp
    apply (rule IT.Lambda)
    apply fast
-  txt \<open>Case @{term Beta}:\<close>
+  txt \<open>Case \<^term>\<open>Beta\<close>:\<close>
   apply atomize
   apply (simp (no_asm_use) add: subst_subst [symmetric])
   apply (rule IT.Beta)