src/HOL/Statespace/StateSpaceEx.thy
changeset 38838 62f6ba39b3d4
parent 29509 1ff0f3f08a7b
child 41959 b460124855b8
--- a/src/HOL/Statespace/StateSpaceEx.thy	Fri Aug 27 22:09:51 2010 +0200
+++ b/src/HOL/Statespace/StateSpaceEx.thy	Fri Aug 27 22:30:25 2010 +0200
@@ -1,14 +1,12 @@
 (*  Title:      StateSpaceEx.thy
-    ID:         $Id$
     Author:     Norbert Schirmer, TU Muenchen
 *)
 
 header {* Examples \label{sec:Examples} *}
 theory StateSpaceEx
 imports StateSpaceLocale StateSpaceSyntax
+begin
 
-begin
-(* FIXME: Use proper keywords file *)
 (*<*)
 syntax
  "_statespace_updates" :: "('a \<Rightarrow> 'b) \<Rightarrow> updbinds \<Rightarrow> ('a \<Rightarrow> 'b)" ("_\<langle>_\<rangle>" [900,0] 900)