src/HOL/NanoJava/AxSem.thy
changeset 16417 9bc16273c2d4
parent 12934 6003b4f916c0
child 23755 1c4672d130b1
--- a/src/HOL/NanoJava/AxSem.thy	Fri Jun 17 11:35:35 2005 +0200
+++ b/src/HOL/NanoJava/AxSem.thy	Fri Jun 17 16:12:49 2005 +0200
@@ -6,7 +6,7 @@
 
 header "Axiomatic Semantics"
 
-theory AxSem = State:
+theory AxSem imports State begin
 
 types assn   = "state => bool"
      vassn   = "val => assn"