src/HOL/NanoJava/OpSem.thy
changeset 16417 9bc16273c2d4
parent 11772 cf618fe8facd
child 23755 1c4672d130b1
--- a/src/HOL/NanoJava/OpSem.thy	Fri Jun 17 11:35:35 2005 +0200
+++ b/src/HOL/NanoJava/OpSem.thy	Fri Jun 17 16:12:49 2005 +0200
@@ -6,7 +6,7 @@
 
 header "Operational Evaluation Semantics"
 
-theory OpSem = State:
+theory OpSem imports State begin
 
 consts
  exec :: "(state \<times> stmt       \<times> nat \<times> state) set"