changeset 3134 | 301b74fcd614 |
parent 3085 | 25d813c5042d |
child 3157 | de89c95c5377 |
--- a/Nominal/Ex/Lambda.thy Wed Mar 14 15:41:54 2012 +0000 +++ b/Nominal/Ex/Lambda.thy Sat Mar 17 05:13:59 2012 +0000 @@ -887,7 +887,7 @@ text {* tests of functions containing if and case *} -(*consts P :: "lam \<Rightarrow> bool" +consts P :: "lam \<Rightarrow> bool" nominal_primrec A :: "lam => lam" @@ -924,7 +924,7 @@ apply(perm_simp) apply(rule allI) apply(rule refl) -oops*) +oops end