src/HOL/Statespace/StateSpaceEx.thy
changeset 29235 2d62b637fa80
parent 28611 983c1855a7af
child 29247 95d3a82857e5
--- a/src/HOL/Statespace/StateSpaceEx.thy	Mon Dec 15 18:12:52 2008 +0100
+++ b/src/HOL/Statespace/StateSpaceEx.thy	Tue Dec 16 15:09:12 2008 +0100
@@ -37,7 +37,7 @@
 projection~/ injection functions that convert from abstract values to
 @{typ "nat"} and @{text "bool"}. The logical content of the locale is: *}
 
-locale vars' =
+class_locale vars' =
   fixes n::'name and b::'name
   assumes "distinct [n, b]" 
 
@@ -204,7 +204,7 @@
   assumes "foo f a b c p1 i1 p2 i2 p3 i3 p4 i4"
   shows True
 proof
-  interpret foo [f a b c p1 i1 p2 i2 p3 i3 p4 i4] by fact
+  class_interpret foo [f a b c p1 i1 p2 i2 p3 i3 p4 i4] by fact
   term "s<a := i>\<cdot>a = i"
 qed