src/HOL/Induct/ABexp.thy
changeset 16417 9bc16273c2d4
parent 14981 e73f8140af78
child 36862 952b2b102a0a
--- a/src/HOL/Induct/ABexp.thy	Fri Jun 17 11:35:35 2005 +0200
+++ b/src/HOL/Induct/ABexp.thy	Fri Jun 17 16:12:49 2005 +0200
@@ -5,7 +5,7 @@
 
 header {* Arithmetic and boolean expressions *}
 
-theory ABexp = Main:
+theory ABexp imports Main begin
 
 datatype 'a aexp =
     IF "'a bexp"  "'a aexp"  "'a aexp"