diff -r ff377f9d030a -r 06950f2b4443 Nominal/Ex/CR.thy --- a/Nominal/Ex/CR.thy Thu Dec 22 04:46:37 2011 +0000 +++ b/Nominal/Ex/CR.thy Thu Dec 22 04:47:05 2011 +0000 @@ -1,5 +1,7 @@ (* CR_Takahashi from Nominal1 ported to Nominal2 *) -theory CR imports Nominal2 begin +theory CR +imports "../Nominal2" +begin atom_decl name @@ -86,6 +88,8 @@ bs1[intro, simp]: "M \b* M" | bs2[intro]: "\M1\b* M2; M2 \b M3\ \ M1 \b* M3" +equivariance beta_star + lemma bs3[intro, trans]: assumes "A \b* B" and "B \b* C"