src/HOL/Library/Nested_Environment.thy
changeset 15131 c69542757a4d
parent 14981 e73f8140af78
child 15140 322485b816ac
--- a/src/HOL/Library/Nested_Environment.thy	Mon Aug 16 14:21:54 2004 +0200
+++ b/src/HOL/Library/Nested_Environment.thy	Mon Aug 16 14:22:27 2004 +0200
@@ -5,7 +5,9 @@
 
 header {* Nested environments *}
 
-theory Nested_Environment = Main:
+theory Nested_Environment
+import Main
+begin
 
 text {*
   Consider a partial function @{term [source] "e :: 'a => 'b option"};