src/HOL/Main.thy
changeset 28263 69eaa97e7e96
parent 28228 7ebe8dc06cbb
child 29304 5c71a6da989d
--- a/src/HOL/Main.thy	Wed Sep 17 21:27:08 2008 +0200
+++ b/src/HOL/Main.thy	Wed Sep 17 21:27:14 2008 +0200
@@ -8,8 +8,6 @@
 imports Plain Code_Eval Map Nat_Int_Bij Recdef
 begin
 
-ML {* val HOL_proofs = ! Proofterm.proofs *}
-
 text {* See further \cite{Nipkow-et-al:2002:tutorial} *}
 
 end