src/HOL/IMPP/Natural.thy
changeset 27362 a6dc1769fdda
parent 24178 4ff1dc2aa18d
child 39159 0dec18004e75
--- a/src/HOL/IMPP/Natural.thy	Wed Jun 25 21:25:51 2008 +0200
+++ b/src/HOL/IMPP/Natural.thy	Wed Jun 25 22:01:34 2008 +0200
@@ -17,10 +17,10 @@
   setlocs :: "state => locals => state"
   getlocs :: "state => locals"
   update  :: "state => vname => val => state"     ("_/[_/::=/_]" [900,0,0] 900)
-syntax (* IN Natural.thy *)
-  loc :: "state => locals"    ("_<_>" [75,0] 75)
-translations
-  "s<X>" == "getlocs s X"
+
+abbreviation
+  loc :: "state => locals"  ("_<_>" [75,0] 75) where
+  "s<X> == getlocs s X"
 
 inductive
   evalc :: "[com,state,    state] => bool"  ("<_,_>/ -c-> _" [0,0,  51] 51)