src/HOL/Statespace/StateSpaceEx.thy
changeset 38838 62f6ba39b3d4
parent 29509 1ff0f3f08a7b
child 41959 b460124855b8
equal deleted inserted replaced
38837:b47ee8df7ab4 38838:62f6ba39b3d4
     1 (*  Title:      StateSpaceEx.thy
     1 (*  Title:      StateSpaceEx.thy
     2     ID:         $Id$
       
     3     Author:     Norbert Schirmer, TU Muenchen
     2     Author:     Norbert Schirmer, TU Muenchen
     4 *)
     3 *)
     5 
     4 
     6 header {* Examples \label{sec:Examples} *}
     5 header {* Examples \label{sec:Examples} *}
     7 theory StateSpaceEx
     6 theory StateSpaceEx
     8 imports StateSpaceLocale StateSpaceSyntax
     7 imports StateSpaceLocale StateSpaceSyntax
     9 
       
    10 begin
     8 begin
    11 (* FIXME: Use proper keywords file *)
     9 
    12 (*<*)
    10 (*<*)
    13 syntax
    11 syntax
    14  "_statespace_updates" :: "('a \<Rightarrow> 'b) \<Rightarrow> updbinds \<Rightarrow> ('a \<Rightarrow> 'b)" ("_\<langle>_\<rangle>" [900,0] 900)
    12  "_statespace_updates" :: "('a \<Rightarrow> 'b) \<Rightarrow> updbinds \<Rightarrow> ('a \<Rightarrow> 'b)" ("_\<langle>_\<rangle>" [900,0] 900)
    15 (*>*)
    13 (*>*)
    16 
    14