Comment out examples with 'True' that do not work because function still does not work
authorCezary Kaliszyk <kaliszyk@in.tum.de>
Fri, 19 Aug 2011 11:01:52 +0900
changeset 2995 6d2859aeebba
parent 2994 4ee772b12032
child 2996 aedcf9e5aa3b
Comment out examples with 'True' that do not work because function still does not work
Nominal/Ex/Lambda.thy
--- 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