src/HOL/IMP/Denotational.thy
changeset 52394 fe33d456b36c
parent 52393 ba73041fd5b3
child 52395 7cc3f42930f3
--- a/src/HOL/IMP/Denotational.thy	Wed Jun 19 10:07:36 2013 +0200
+++ b/src/HOL/IMP/Denotational.thy	Wed Jun 19 10:14:50 2013 +0200
@@ -2,7 +2,7 @@
 
 header "Denotational Semantics of Commands"
 
-theory Denotation imports Big_Step begin
+theory Denotational imports Big_Step begin
 
 type_synonym com_den = "(state \<times> state) set"