--- 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"
--- a/src/HOL/ROOT Wed Jun 19 10:07:36 2013 +0200
+++ b/src/HOL/ROOT Wed Jun 19 10:14:50 2013 +0200
@@ -119,7 +119,7 @@
BExp
ASM
Finite_Reachable
- Denotation
+ Denotational
Comp_Rev
Poly_Types
Sec_Typing