removed junk
authorChristian Urban <christian dot urban at kcl dot ac dot uk>
Mon, 20 Jul 2015 11:21:59 +0100
changeset 3242 4af8a92396ce
parent 3240 f80fa0d18d81
child 3243 c4f31f1564b7
child 3244 a44479bde681
removed junk
Nominal/Ex/Lambda.thy
--- a/Nominal/Ex/Lambda.thy	Thu Jul 09 09:12:44 2015 +0100
+++ b/Nominal/Ex/Lambda.thy	Mon Jul 20 11:21:59 2015 +0100
@@ -14,14 +14,6 @@
 
 thm obtain_atom
 
-lemma 
- "(\<forall>thesis. (finite X \<longrightarrow> (\<forall>a. ((a \<notin> X \<and> sort_of a = s) \<longrightarrow> thesis)) \<longrightarrow> thesis)) \<longleftrightarrow>
-  (finite X \<longrightarrow> (\<exists> a. (a \<notin> X \<and> sort_of a = s)))"
-apply(auto) 
-done
-
-
-
 ML {* trace := true *}
 
 nominal_datatype lam =
@@ -996,8 +988,6 @@
 
 text {* tests of functions containing if and case *}
 
-consts P :: "lam \<Rightarrow> bool"
-
 (*
 nominal_function  
   A :: "lam => lam"