src/HOL/Statespace/StateSpaceSyntax.thy
author wenzelm
Thu, 10 Jan 2013 19:53:38 +0100
changeset 50808 1702ed63c2db
parent 41959 b460124855b8
child 52143 36ffe23b25f8
permissions -rw-r--r--
more general prover termination dialog, which might indicate undetected failure or just ML "exit 0";

(*  Title:      HOL/Statespace/StateSpaceSyntax.thy
    Author:     Norbert Schirmer, TU Muenchen
*)

header {* Syntax for State Space Lookup and Update \label{sec:StateSpaceSyntax}*}
theory StateSpaceSyntax
imports StateSpaceLocale
begin

text {* The state space syntax is kept in an extra theory so that you
can choose if you want to use it or not.  *}

syntax 
  "_statespace_lookup" :: "('a \<Rightarrow> 'b) \<Rightarrow> 'a \<Rightarrow> 'c"  ("_\<cdot>_" [60, 60] 60)
  "_statespace_update" :: "('a \<Rightarrow> 'b) \<Rightarrow> 'a \<Rightarrow> 'c \<Rightarrow> ('a \<Rightarrow> 'b)"
  "_statespace_updates" :: "('a \<Rightarrow> 'b) \<Rightarrow> updbinds \<Rightarrow> ('a \<Rightarrow> 'b)"  ("_<_>" [900, 0] 900)

translations
  "_statespace_updates f (_updbinds b bs)" ==
    "_statespace_updates (_statespace_updates f b) bs"
  "s<x:=y>" == "_statespace_update s x y"


parse_translation (advanced)
{*
 [(@{syntax_const "_statespace_lookup"}, StateSpace.lookup_tr),
  (@{syntax_const "_statespace_update"}, StateSpace.update_tr)]
*}


print_translation (advanced)
{*
 [(@{const_syntax lookup}, StateSpace.lookup_tr'),
  (@{const_syntax update}, StateSpace.update_tr')]
*}

end