Quot/Nominal/LFex.thy
changeset 1021 bacf3584640e
parent 1004 44b013c59653
child 1022 cc5830c452c4
--- a/Quot/Nominal/LFex.thy	Tue Feb 02 09:51:39 2010 +0100
+++ b/Quot/Nominal/LFex.thy	Tue Feb 02 10:20:54 2010 +0100
@@ -17,7 +17,6 @@
   | Var "name"
   | App "trm" "trm"
   | Lam "ty" "name" "trm"
-print_theorems
 
 primrec
     rfv_kind :: "kind \<Rightarrow> atom set"
@@ -33,7 +32,6 @@
 | "rfv_trm (Var x) = {atom x}"
 | "rfv_trm (App M N) = (rfv_trm M) \<union> (rfv_trm N)"
 | "rfv_trm (Lam A x M) = (rfv_ty A) \<union> ((rfv_trm M) - {atom x})"
-print_theorems
 
 instantiation kind and ty and trm :: pt
 begin