src/Pure/Pure.thy
changeset 26426 ddac7ef1e991
parent 23824 8ad7131dbfcf
child 26435 bdce320cd426
--- a/src/Pure/Pure.thy	Thu Mar 27 14:41:10 2008 +0100
+++ b/src/Pure/Pure.thy	Thu Mar 27 14:41:12 2008 +0100
@@ -2,11 +2,7 @@
     ID:         $Id$
 *)
 
-header {* The Pure theory *}
-
-theory Pure
-imports ProtoPure
-begin
+section {* The Pure theory *}
 
 setup  -- {* Common setup of internal components *}
 
@@ -103,4 +99,3 @@
   qed
 qed
 
-end