src/HOL/IMP/Denotation.thy
changeset 16417 9bc16273c2d4
parent 15481 fc075ae929e4
child 18372 2bffdf62fe7f
--- a/src/HOL/IMP/Denotation.thy	Fri Jun 17 11:35:35 2005 +0200
+++ b/src/HOL/IMP/Denotation.thy	Fri Jun 17 16:12:49 2005 +0200
@@ -6,7 +6,7 @@
 
 header "Denotational Semantics of Commands"
 
-theory Denotation = Natural:
+theory Denotation imports Natural begin
 
 types com_den = "(state\<times>state)set"