products/sources/formale sprachen/Isabelle/HOL/Statespace image not shown  

Quellcode-Bibliothek

© Kompilation durch diese Firma

[Weder Korrektheit noch Funktionsfähigkeit der Software werden zugesichert.]

Datei: StateSpaceSyntax.thy   Sprache: Isabelle

Original von: Isabelle©

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


section \<open>Syntax for State Space Lookup and Update \label{sec:StateSpaceSyntax}\<close>
theory StateSpaceSyntax
imports StateSpaceLocale
begin

text \<open>The state space syntax is kept in an extra theory so that you
can choose if you want to use it or not.\<close>

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

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


parse_translation
\<open>
 [(\<^syntax_const>\<open>_statespace_lookup\<close>, StateSpace.lookup_tr),
  (\<^syntax_const>\<open>_statespace_update\<close>, StateSpace.update_tr)]
\<close>


print_translation
\<open>
 [(\<^const_syntax>\<open>lookup\<close>, StateSpace.lookup_tr'),
  (\<^const_syntax>\<open>update\<close>, StateSpace.update_tr')]
\<close>

end

¤ Dauer der Verarbeitung: 0.0 Sekunden  (vorverarbeitet)  ¤





Kontakt
Drucken
Kontakt
sprechenden Kalenders

in der Quellcodebibliothek suchen




schauen Sie vor die Tür

Fenster


Die Firma ist wie angegeben erreichbar.

Die farbliche Syntaxdarstellung ist noch experimentell.


Bot Zugriff