diff -r 143f58bb34f9 -r 0909deb8059b src/HOL/Nominal/Examples/Class3.thy --- a/src/HOL/Nominal/Examples/Class3.thy Thu May 26 16:57:14 2016 +0200 +++ b/src/HOL/Nominal/Examples/Class3.thy Thu May 26 17:51:22 2016 +0200 @@ -2,7 +2,7 @@ imports Class2 begin -text {* 3rd Main Lemma *} +text \3rd Main Lemma\ lemma Cut_a_redu_elim: assumes a: "Cut .M (x).N \\<^sub>a R" @@ -2246,7 +2246,7 @@ apply(blast)+ done -text {* helper-stuff to set up the induction *} +text \helper-stuff to set up the induction\ abbreviation SNa_set :: "trm set" @@ -2359,7 +2359,7 @@ apply(simp add: alpha fresh_prod fresh_atm) done -text {* 3rd lemma *} +text \3rd lemma\ lemma CUT_SNa_aux: assumes a1: ":M \ (\\)" @@ -4927,7 +4927,7 @@ done -text {* typing relation *} +text \typing relation\ inductive typing :: "ctxtn \ trm \ ctxtc \ bool" ("_ \ _ \ _" [100,100,100] 100)