src/HOL/Library/Open_State_Syntax.thy
author wenzelm
Sun, 24 Dec 2023 13:20:40 +0100
changeset 79353 af7881b2299d
parent 72581 de581f98a3a1
child 80783 14ed085de388
permissions -rw-r--r--
tuned names;
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
66270
403d84138c5c State_Monad ~> Open_State_Syntax
Lars Hupel <lars.hupel@mytum.de>
parents: 66258
diff changeset
     1
(*  Title:      HOL/Library/Open_State_Syntax.thy
21192
5fe5cd5fede7 added state monad to HOL library
haftmann
parents:
diff changeset
     2
    Author:     Florian Haftmann, TU Muenchen
5fe5cd5fede7 added state monad to HOL library
haftmann
parents:
diff changeset
     3
*)
5fe5cd5fede7 added state monad to HOL library
haftmann
parents:
diff changeset
     4
60500
903bb1495239 isabelle update_cartouches;
wenzelm
parents: 58881
diff changeset
     5
section \<open>Combinator syntax for generic, open state monads (single-threaded monads)\<close>
21192
5fe5cd5fede7 added state monad to HOL library
haftmann
parents:
diff changeset
     6
66270
403d84138c5c State_Monad ~> Open_State_Syntax
Lars Hupel <lars.hupel@mytum.de>
parents: 66258
diff changeset
     7
theory Open_State_Syntax
66258
2b83dd24b301 dropped superfluous theory imports
haftmann
parents: 63680
diff changeset
     8
imports Main
21192
5fe5cd5fede7 added state monad to HOL library
haftmann
parents:
diff changeset
     9
begin
5fe5cd5fede7 added state monad to HOL library
haftmann
parents:
diff changeset
    10
72581
de581f98a3a1 bundled syntax for state monad combinators
haftmann
parents: 69593
diff changeset
    11
context
de581f98a3a1 bundled syntax for state monad combinators
haftmann
parents: 69593
diff changeset
    12
  includes state_combinator_syntax
de581f98a3a1 bundled syntax for state monad combinators
haftmann
parents: 69593
diff changeset
    13
begin
de581f98a3a1 bundled syntax for state monad combinators
haftmann
parents: 69593
diff changeset
    14
60500
903bb1495239 isabelle update_cartouches;
wenzelm
parents: 58881
diff changeset
    15
subsection \<open>Motivation\<close>
21192
5fe5cd5fede7 added state monad to HOL library
haftmann
parents:
diff changeset
    16
60500
903bb1495239 isabelle update_cartouches;
wenzelm
parents: 58881
diff changeset
    17
text \<open>
40359
84388bba911d dropped return abbreviation for Pair -- confusing if combined with monad syntax; tuned document
haftmann
parents: 38345
diff changeset
    18
  The logic HOL has no notion of constructor classes, so it is not
84388bba911d dropped return abbreviation for Pair -- confusing if combined with monad syntax; tuned document
haftmann
parents: 38345
diff changeset
    19
  possible to model monads the Haskell way in full genericity in
84388bba911d dropped return abbreviation for Pair -- confusing if combined with monad syntax; tuned document
haftmann
parents: 38345
diff changeset
    20
  Isabelle/HOL.
21192
5fe5cd5fede7 added state monad to HOL library
haftmann
parents:
diff changeset
    21
  
40359
84388bba911d dropped return abbreviation for Pair -- confusing if combined with monad syntax; tuned document
haftmann
parents: 38345
diff changeset
    22
  However, this theory provides substantial support for a very common
84388bba911d dropped return abbreviation for Pair -- confusing if combined with monad syntax; tuned document
haftmann
parents: 38345
diff changeset
    23
  class of monads: \emph{state monads} (or \emph{single-threaded
84388bba911d dropped return abbreviation for Pair -- confusing if combined with monad syntax; tuned document
haftmann
parents: 38345
diff changeset
    24
  monads}, since a state is transformed single-threadedly).
21192
5fe5cd5fede7 added state monad to HOL library
haftmann
parents:
diff changeset
    25
5fe5cd5fede7 added state monad to HOL library
haftmann
parents:
diff changeset
    26
  To enter from the Haskell world,
68224
1f7308050349 prefer HTTPS;
wenzelm
parents: 67399
diff changeset
    27
  \<^url>\<open>https://www.engr.mun.ca/~theo/Misc/haskell_and_monads.htm\<close> makes
40359
84388bba911d dropped return abbreviation for Pair -- confusing if combined with monad syntax; tuned document
haftmann
parents: 38345
diff changeset
    28
  a good motivating start.  Here we just sketch briefly how those
84388bba911d dropped return abbreviation for Pair -- confusing if combined with monad syntax; tuned document
haftmann
parents: 38345
diff changeset
    29
  monads enter the game of Isabelle/HOL.
60500
903bb1495239 isabelle update_cartouches;
wenzelm
parents: 58881
diff changeset
    30
\<close>
21192
5fe5cd5fede7 added state monad to HOL library
haftmann
parents:
diff changeset
    31
60500
903bb1495239 isabelle update_cartouches;
wenzelm
parents: 58881
diff changeset
    32
subsection \<open>State transformations and combinators\<close>
21192
5fe5cd5fede7 added state monad to HOL library
haftmann
parents:
diff changeset
    33
60500
903bb1495239 isabelle update_cartouches;
wenzelm
parents: 58881
diff changeset
    34
text \<open>
21192
5fe5cd5fede7 added state monad to HOL library
haftmann
parents:
diff changeset
    35
  We classify functions operating on states into two categories:
5fe5cd5fede7 added state monad to HOL library
haftmann
parents:
diff changeset
    36
5fe5cd5fede7 added state monad to HOL library
haftmann
parents:
diff changeset
    37
  \begin{description}
40359
84388bba911d dropped return abbreviation for Pair -- confusing if combined with monad syntax; tuned document
haftmann
parents: 38345
diff changeset
    38
61585
a9599d3d7610 isabelle update_cartouches -c -t;
wenzelm
parents: 60500
diff changeset
    39
    \item[transformations] with type signature \<open>\<sigma> \<Rightarrow> \<sigma>'\<close>,
21192
5fe5cd5fede7 added state monad to HOL library
haftmann
parents:
diff changeset
    40
      transforming a state.
40359
84388bba911d dropped return abbreviation for Pair -- confusing if combined with monad syntax; tuned document
haftmann
parents: 38345
diff changeset
    41
61585
a9599d3d7610 isabelle update_cartouches -c -t;
wenzelm
parents: 60500
diff changeset
    42
    \item[``yielding'' transformations] with type signature \<open>\<sigma>
a9599d3d7610 isabelle update_cartouches -c -t;
wenzelm
parents: 60500
diff changeset
    43
      \<Rightarrow> \<alpha> \<times> \<sigma>'\<close>, ``yielding'' a side result while transforming a
40359
84388bba911d dropped return abbreviation for Pair -- confusing if combined with monad syntax; tuned document
haftmann
parents: 38345
diff changeset
    44
      state.
84388bba911d dropped return abbreviation for Pair -- confusing if combined with monad syntax; tuned document
haftmann
parents: 38345
diff changeset
    45
61585
a9599d3d7610 isabelle update_cartouches -c -t;
wenzelm
parents: 60500
diff changeset
    46
    \item[queries] with type signature \<open>\<sigma> \<Rightarrow> \<alpha>\<close>, computing a
40359
84388bba911d dropped return abbreviation for Pair -- confusing if combined with monad syntax; tuned document
haftmann
parents: 38345
diff changeset
    47
      result dependent on a state.
84388bba911d dropped return abbreviation for Pair -- confusing if combined with monad syntax; tuned document
haftmann
parents: 38345
diff changeset
    48
21192
5fe5cd5fede7 added state monad to HOL library
haftmann
parents:
diff changeset
    49
  \end{description}
5fe5cd5fede7 added state monad to HOL library
haftmann
parents:
diff changeset
    50
61585
a9599d3d7610 isabelle update_cartouches -c -t;
wenzelm
parents: 60500
diff changeset
    51
  By convention we write \<open>\<sigma>\<close> for types representing states and
a9599d3d7610 isabelle update_cartouches -c -t;
wenzelm
parents: 60500
diff changeset
    52
  \<open>\<alpha>\<close>, \<open>\<beta>\<close>, \<open>\<gamma>\<close>, \<open>\<dots>\<close> for types
40359
84388bba911d dropped return abbreviation for Pair -- confusing if combined with monad syntax; tuned document
haftmann
parents: 38345
diff changeset
    53
  representing side results.  Type changes due to transformations are
84388bba911d dropped return abbreviation for Pair -- confusing if combined with monad syntax; tuned document
haftmann
parents: 38345
diff changeset
    54
  not excluded in our scenario.
21192
5fe5cd5fede7 added state monad to HOL library
haftmann
parents:
diff changeset
    55
61585
a9599d3d7610 isabelle update_cartouches -c -t;
wenzelm
parents: 60500
diff changeset
    56
  We aim to assert that values of any state type \<open>\<sigma>\<close> are used
40359
84388bba911d dropped return abbreviation for Pair -- confusing if combined with monad syntax; tuned document
haftmann
parents: 38345
diff changeset
    57
  in a single-threaded way: after application of a transformation on a
61585
a9599d3d7610 isabelle update_cartouches -c -t;
wenzelm
parents: 60500
diff changeset
    58
  value of type \<open>\<sigma>\<close>, the former value should not be used
40359
84388bba911d dropped return abbreviation for Pair -- confusing if combined with monad syntax; tuned document
haftmann
parents: 38345
diff changeset
    59
  again.  To achieve this, we use a set of monad combinators:
60500
903bb1495239 isabelle update_cartouches;
wenzelm
parents: 58881
diff changeset
    60
\<close>
21192
5fe5cd5fede7 added state monad to HOL library
haftmann
parents:
diff changeset
    61
60500
903bb1495239 isabelle update_cartouches;
wenzelm
parents: 58881
diff changeset
    62
text \<open>
69593
3dda49e08b9d isabelle update -u control_cartouches;
wenzelm
parents: 68224
diff changeset
    63
  Given two transformations \<^term>\<open>f\<close> and \<^term>\<open>g\<close>, they may be
3dda49e08b9d isabelle update -u control_cartouches;
wenzelm
parents: 68224
diff changeset
    64
  directly composed using the \<^term>\<open>(\<circ>>)\<close> combinator, forming a
3dda49e08b9d isabelle update -u control_cartouches;
wenzelm
parents: 68224
diff changeset
    65
  forward composition: \<^prop>\<open>(f \<circ>> g) s = f (g s)\<close>.
21192
5fe5cd5fede7 added state monad to HOL library
haftmann
parents:
diff changeset
    66
5fe5cd5fede7 added state monad to HOL library
haftmann
parents:
diff changeset
    67
  After any yielding transformation, we bind the side result
40359
84388bba911d dropped return abbreviation for Pair -- confusing if combined with monad syntax; tuned document
haftmann
parents: 38345
diff changeset
    68
  immediately using a lambda abstraction.  This is the purpose of the
69593
3dda49e08b9d isabelle update -u control_cartouches;
wenzelm
parents: 68224
diff changeset
    69
  \<^term>\<open>(\<circ>\<rightarrow>)\<close> combinator: \<^prop>\<open>(f \<circ>\<rightarrow> (\<lambda>x. g)) s = (let (x, s')
3dda49e08b9d isabelle update -u control_cartouches;
wenzelm
parents: 68224
diff changeset
    70
  = f s in g s')\<close>.
21192
5fe5cd5fede7 added state monad to HOL library
haftmann
parents:
diff changeset
    71
69593
3dda49e08b9d isabelle update -u control_cartouches;
wenzelm
parents: 68224
diff changeset
    72
  For queries, the existing \<^term>\<open>Let\<close> is appropriate.
21192
5fe5cd5fede7 added state monad to HOL library
haftmann
parents:
diff changeset
    73
40359
84388bba911d dropped return abbreviation for Pair -- confusing if combined with monad syntax; tuned document
haftmann
parents: 38345
diff changeset
    74
  Naturally, a computation may yield a side result by pairing it to
84388bba911d dropped return abbreviation for Pair -- confusing if combined with monad syntax; tuned document
haftmann
parents: 38345
diff changeset
    75
  the state from the left; we introduce the suggestive abbreviation
69593
3dda49e08b9d isabelle update -u control_cartouches;
wenzelm
parents: 68224
diff changeset
    76
  \<^term>\<open>return\<close> for this purpose.
21192
5fe5cd5fede7 added state monad to HOL library
haftmann
parents:
diff changeset
    77
40359
84388bba911d dropped return abbreviation for Pair -- confusing if combined with monad syntax; tuned document
haftmann
parents: 38345
diff changeset
    78
  The most crucial distinction to Haskell is that we do not need to
84388bba911d dropped return abbreviation for Pair -- confusing if combined with monad syntax; tuned document
haftmann
parents: 38345
diff changeset
    79
  introduce distinguished type constructors for different kinds of
84388bba911d dropped return abbreviation for Pair -- confusing if combined with monad syntax; tuned document
haftmann
parents: 38345
diff changeset
    80
  state.  This has two consequences:
84388bba911d dropped return abbreviation for Pair -- confusing if combined with monad syntax; tuned document
haftmann
parents: 38345
diff changeset
    81
21192
5fe5cd5fede7 added state monad to HOL library
haftmann
parents:
diff changeset
    82
  \begin{itemize}
40359
84388bba911d dropped return abbreviation for Pair -- confusing if combined with monad syntax; tuned document
haftmann
parents: 38345
diff changeset
    83
84388bba911d dropped return abbreviation for Pair -- confusing if combined with monad syntax; tuned document
haftmann
parents: 38345
diff changeset
    84
    \item The monad model does not state anything about the kind of
84388bba911d dropped return abbreviation for Pair -- confusing if combined with monad syntax; tuned document
haftmann
parents: 38345
diff changeset
    85
       state; the model for the state is completely orthogonal and may
84388bba911d dropped return abbreviation for Pair -- confusing if combined with monad syntax; tuned document
haftmann
parents: 38345
diff changeset
    86
       be specified completely independently.
84388bba911d dropped return abbreviation for Pair -- confusing if combined with monad syntax; tuned document
haftmann
parents: 38345
diff changeset
    87
84388bba911d dropped return abbreviation for Pair -- confusing if combined with monad syntax; tuned document
haftmann
parents: 38345
diff changeset
    88
    \item There is no distinguished type constructor encapsulating
84388bba911d dropped return abbreviation for Pair -- confusing if combined with monad syntax; tuned document
haftmann
parents: 38345
diff changeset
    89
       away the state transformation, i.e.~transformations may be
84388bba911d dropped return abbreviation for Pair -- confusing if combined with monad syntax; tuned document
haftmann
parents: 38345
diff changeset
    90
       applied directly without using any lifting or providing and
84388bba911d dropped return abbreviation for Pair -- confusing if combined with monad syntax; tuned document
haftmann
parents: 38345
diff changeset
    91
       dropping units (``open monad'').
84388bba911d dropped return abbreviation for Pair -- confusing if combined with monad syntax; tuned document
haftmann
parents: 38345
diff changeset
    92
21192
5fe5cd5fede7 added state monad to HOL library
haftmann
parents:
diff changeset
    93
    \item The type of states may change due to a transformation.
40359
84388bba911d dropped return abbreviation for Pair -- confusing if combined with monad syntax; tuned document
haftmann
parents: 38345
diff changeset
    94
21192
5fe5cd5fede7 added state monad to HOL library
haftmann
parents:
diff changeset
    95
  \end{itemize}
60500
903bb1495239 isabelle update_cartouches;
wenzelm
parents: 58881
diff changeset
    96
\<close>
21192
5fe5cd5fede7 added state monad to HOL library
haftmann
parents:
diff changeset
    97
5fe5cd5fede7 added state monad to HOL library
haftmann
parents:
diff changeset
    98
60500
903bb1495239 isabelle update_cartouches;
wenzelm
parents: 58881
diff changeset
    99
subsection \<open>Monad laws\<close>
21192
5fe5cd5fede7 added state monad to HOL library
haftmann
parents:
diff changeset
   100
60500
903bb1495239 isabelle update_cartouches;
wenzelm
parents: 58881
diff changeset
   101
text \<open>
40359
84388bba911d dropped return abbreviation for Pair -- confusing if combined with monad syntax; tuned document
haftmann
parents: 38345
diff changeset
   102
  The common monadic laws hold and may also be used as normalization
84388bba911d dropped return abbreviation for Pair -- confusing if combined with monad syntax; tuned document
haftmann
parents: 38345
diff changeset
   103
  rules for monadic expressions:
60500
903bb1495239 isabelle update_cartouches;
wenzelm
parents: 58881
diff changeset
   104
\<close>
21192
5fe5cd5fede7 added state monad to HOL library
haftmann
parents:
diff changeset
   105
28145
af3923ed4786 dropped "run" marker in monad syntax
haftmann
parents: 27487
diff changeset
   106
lemmas monad_simp = Pair_scomp scomp_Pair id_fcomp fcomp_id
af3923ed4786 dropped "run" marker in monad syntax
haftmann
parents: 27487
diff changeset
   107
  scomp_scomp scomp_fcomp fcomp_scomp fcomp_assoc
21192
5fe5cd5fede7 added state monad to HOL library
haftmann
parents:
diff changeset
   108
60500
903bb1495239 isabelle update_cartouches;
wenzelm
parents: 58881
diff changeset
   109
text \<open>
21192
5fe5cd5fede7 added state monad to HOL library
haftmann
parents:
diff changeset
   110
  Evaluation of monadic expressions by force:
60500
903bb1495239 isabelle update_cartouches;
wenzelm
parents: 58881
diff changeset
   111
\<close>
21192
5fe5cd5fede7 added state monad to HOL library
haftmann
parents:
diff changeset
   112
28145
af3923ed4786 dropped "run" marker in monad syntax
haftmann
parents: 27487
diff changeset
   113
lemmas monad_collapse = monad_simp fcomp_apply scomp_apply split_beta
26260
haftmann
parents: 26141
diff changeset
   114
72581
de581f98a3a1 bundled syntax for state monad combinators
haftmann
parents: 69593
diff changeset
   115
end
de581f98a3a1 bundled syntax for state monad combinators
haftmann
parents: 69593
diff changeset
   116
37817
71e5546b1965 tuned infix syntax
haftmann
parents: 37791
diff changeset
   117
60500
903bb1495239 isabelle update_cartouches;
wenzelm
parents: 58881
diff changeset
   118
subsection \<open>Do-syntax\<close>
37817
71e5546b1965 tuned infix syntax
haftmann
parents: 37791
diff changeset
   119
41229
d797baa3d57c replaced command 'nonterminals' by slightly modernized version 'nonterminal';
wenzelm
parents: 40361
diff changeset
   120
nonterminal sdo_binds and sdo_bind
37932
d00a3f47b607 more generous memory settings for scala check
haftmann
parents: 37817
diff changeset
   121
d00a3f47b607 more generous memory settings for scala check
haftmann
parents: 37817
diff changeset
   122
syntax
d00a3f47b607 more generous memory settings for scala check
haftmann
parents: 37817
diff changeset
   123
  "_sdo_block" :: "sdo_binds \<Rightarrow> 'a" ("exec {//(2  _)//}" [12] 62)
61955
e96292f32c3c former "xsymbols" syntax is used by default, and ASCII replacement syntax with print mode "ASCII";
wenzelm
parents: 61585
diff changeset
   124
  "_sdo_bind"  :: "[pttrn, 'a] \<Rightarrow> sdo_bind" ("(_ \<leftarrow>/ _)" 13)
37932
d00a3f47b607 more generous memory settings for scala check
haftmann
parents: 37817
diff changeset
   125
  "_sdo_let" :: "[pttrn, 'a] \<Rightarrow> sdo_bind" ("(2let _ =/ _)" [1000, 13] 13)
d00a3f47b607 more generous memory settings for scala check
haftmann
parents: 37817
diff changeset
   126
  "_sdo_then" :: "'a \<Rightarrow> sdo_bind" ("_" [14] 13)
d00a3f47b607 more generous memory settings for scala check
haftmann
parents: 37817
diff changeset
   127
  "_sdo_final" :: "'a \<Rightarrow> sdo_binds" ("_")
d00a3f47b607 more generous memory settings for scala check
haftmann
parents: 37817
diff changeset
   128
  "_sdo_cons" :: "[sdo_bind, sdo_binds] \<Rightarrow> sdo_binds" ("_;//_" [13, 12] 12)
21192
5fe5cd5fede7 added state monad to HOL library
haftmann
parents:
diff changeset
   129
61955
e96292f32c3c former "xsymbols" syntax is used by default, and ASCII replacement syntax with print mode "ASCII";
wenzelm
parents: 61585
diff changeset
   130
syntax (ASCII)
e96292f32c3c former "xsymbols" syntax is used by default, and ASCII replacement syntax with print mode "ASCII";
wenzelm
parents: 61585
diff changeset
   131
  "_sdo_bind" :: "[pttrn, 'a] \<Rightarrow> sdo_bind" ("(_ <-/ _)" 13)
37932
d00a3f47b607 more generous memory settings for scala check
haftmann
parents: 37817
diff changeset
   132
d00a3f47b607 more generous memory settings for scala check
haftmann
parents: 37817
diff changeset
   133
translations
d00a3f47b607 more generous memory settings for scala check
haftmann
parents: 37817
diff changeset
   134
  "_sdo_block (_sdo_cons (_sdo_bind p t) (_sdo_final e))"
d00a3f47b607 more generous memory settings for scala check
haftmann
parents: 37817
diff changeset
   135
    == "CONST scomp t (\<lambda>p. e)"
d00a3f47b607 more generous memory settings for scala check
haftmann
parents: 37817
diff changeset
   136
  "_sdo_block (_sdo_cons (_sdo_then t) (_sdo_final e))"
38345
8b8fc27c1872 print fcomp combinator only monadic in connection with other monadic expressions
haftmann
parents: 37932
diff changeset
   137
    => "CONST fcomp t e"
8b8fc27c1872 print fcomp combinator only monadic in connection with other monadic expressions
haftmann
parents: 37932
diff changeset
   138
  "_sdo_final (_sdo_block (_sdo_cons (_sdo_then t) (_sdo_final e)))"
8b8fc27c1872 print fcomp combinator only monadic in connection with other monadic expressions
haftmann
parents: 37932
diff changeset
   139
    <= "_sdo_final (CONST fcomp t e)"
8b8fc27c1872 print fcomp combinator only monadic in connection with other monadic expressions
haftmann
parents: 37932
diff changeset
   140
  "_sdo_block (_sdo_cons (_sdo_then t) e)"
8b8fc27c1872 print fcomp combinator only monadic in connection with other monadic expressions
haftmann
parents: 37932
diff changeset
   141
    <= "CONST fcomp t (_sdo_block e)"
37932
d00a3f47b607 more generous memory settings for scala check
haftmann
parents: 37817
diff changeset
   142
  "_sdo_block (_sdo_cons (_sdo_let p t) bs)"
d00a3f47b607 more generous memory settings for scala check
haftmann
parents: 37817
diff changeset
   143
    == "let p = t in _sdo_block bs"
d00a3f47b607 more generous memory settings for scala check
haftmann
parents: 37817
diff changeset
   144
  "_sdo_block (_sdo_cons b (_sdo_cons c cs))"
d00a3f47b607 more generous memory settings for scala check
haftmann
parents: 37817
diff changeset
   145
    == "_sdo_block (_sdo_cons b (_sdo_final (_sdo_block (_sdo_cons c cs))))"
d00a3f47b607 more generous memory settings for scala check
haftmann
parents: 37817
diff changeset
   146
  "_sdo_cons (_sdo_let p t) (_sdo_final s)"
d00a3f47b607 more generous memory settings for scala check
haftmann
parents: 37817
diff changeset
   147
    == "_sdo_final (let p = t in s)"
d00a3f47b607 more generous memory settings for scala check
haftmann
parents: 37817
diff changeset
   148
  "_sdo_block (_sdo_final e)" => "e"
37817
71e5546b1965 tuned infix syntax
haftmann
parents: 37791
diff changeset
   149
60500
903bb1495239 isabelle update_cartouches;
wenzelm
parents: 58881
diff changeset
   150
text \<open>
63680
6e1e8b5abbfa more symbols;
wenzelm
parents: 63362
diff changeset
   151
  For an example, see \<^file>\<open>~~/src/HOL/Proofs/Extraction/Higman_Extraction.thy\<close>.
60500
903bb1495239 isabelle update_cartouches;
wenzelm
parents: 58881
diff changeset
   152
\<close>
21192
5fe5cd5fede7 added state monad to HOL library
haftmann
parents:
diff changeset
   153
22664
e965391e2864 do translation: CONST;
wenzelm
parents: 22492
diff changeset
   154
end