Nominal/Ex/Lambda.thy
changeset 2995 6d2859aeebba
parent 2982 4a00077c008f
child 3046 9b0324e1293b
child 3071 11f6a561eb4b
--- a/Nominal/Ex/Lambda.thy	Fri Aug 19 10:56:12 2011 +0900
+++ b/Nominal/Ex/Lambda.thy	Fri Aug 19 11:01:52 2011 +0900
@@ -886,7 +886,7 @@
 
 text {* tests of functions containing if and case *}
 
-consts P :: "lam \<Rightarrow> bool"
+(*consts P :: "lam \<Rightarrow> bool"
 
 nominal_primrec  
   A :: "lam => lam"
@@ -923,7 +923,7 @@
 apply(perm_simp)
 apply(rule allI)
 apply(rule refl)
-oops
+oops*)
 
 end