| author | wenzelm | 
| Wed, 02 May 2012 22:37:50 +0200 | |
| changeset 47863 | ec5d54029664 | 
| parent 46143 | c932c80d3eae | 
| child 52622 | e0ff1625e96d | 
| permissions | -rw-r--r-- | 
| 37790 | 1 | (* Author: Alexander Krauss, TU Muenchen | 
| 2 | Author: Christian Sternagel, University of Innsbruck | |
| 3 | *) | |
| 4 | ||
| 5 | header {* Monad notation for arbitrary types *}
 | |
| 6 | ||
| 7 | theory Monad_Syntax | |
| 45990 
b7b905b23b2a
incorporated More_Set and More_List into the Main body -- to be consolidated later
 haftmann parents: 
45964diff
changeset | 8 | imports Main "~~/src/Tools/Adhoc_Overloading" | 
| 37790 | 9 | begin | 
| 10 | ||
| 37791 | 11 | text {*
 | 
| 12 | We provide a convenient do-notation for monadic expressions | |
| 13 |   well-known from Haskell.  @{const Let} is printed
 | |
| 14 | specially in do-expressions. | |
| 15 | *} | |
| 16 | ||
| 37790 | 17 | consts | 
| 37816 | 18 | bind :: "['a, 'b \<Rightarrow> 'c] \<Rightarrow> 'c" (infixr ">>=" 54) | 
| 37790 | 19 | |
| 20 | notation (xsymbols) | |
| 37816 | 21 | bind (infixr "\<guillemotright>=" 54) | 
| 37790 | 22 | |
| 37848 | 23 | notation (latex output) | 
| 24 | bind (infixr "\<bind>" 54) | |
| 25 | ||
| 37790 | 26 | abbreviation (do_notation) | 
| 37816 | 27 | bind_do :: "['a, 'b \<Rightarrow> 'c] \<Rightarrow> 'c" | 
| 37790 | 28 | where | 
| 37816 | 29 | "bind_do \<equiv> bind" | 
| 37790 | 30 | |
| 31 | notation (output) | |
| 37816 | 32 | bind_do (infixr ">>=" 54) | 
| 37790 | 33 | |
| 34 | notation (xsymbols output) | |
| 37816 | 35 | bind_do (infixr "\<guillemotright>=" 54) | 
| 37790 | 36 | |
| 37848 | 37 | notation (latex output) | 
| 38 | bind_do (infixr "\<bind>" 54) | |
| 39 | ||
| 41229 
d797baa3d57c
replaced command 'nonterminals' by slightly modernized version 'nonterminal';
 wenzelm parents: 
39151diff
changeset | 40 | nonterminal do_binds and do_bind | 
| 37790 | 41 | |
| 42 | syntax | |
| 43 |   "_do_block" :: "do_binds \<Rightarrow> 'a" ("do {//(2  _)//}" [12] 62)
 | |
| 44 |   "_do_bind" :: "[pttrn, 'a] \<Rightarrow> do_bind" ("(_ <-/ _)" 13)
 | |
| 45 |   "_do_let" :: "[pttrn, 'a] \<Rightarrow> do_bind" ("(2let _ =/ _)" [1000, 13] 13)
 | |
| 46 |   "_do_then" :: "'a \<Rightarrow> do_bind" ("_" [14] 13)
 | |
| 47 |   "_do_final" :: "'a \<Rightarrow> do_binds" ("_")
 | |
| 48 |   "_do_cons" :: "[do_bind, do_binds] \<Rightarrow> do_binds" ("_;//_" [13, 12] 12)
 | |
| 49 | "_thenM" :: "['a, 'b] \<Rightarrow> 'b" (infixr ">>" 54) | |
| 50 | ||
| 51 | syntax (xsymbols) | |
| 52 |   "_do_bind"  :: "[pttrn, 'a] \<Rightarrow> do_bind" ("(_ \<leftarrow>/ _)" 13)
 | |
| 53 | "_thenM" :: "['a, 'b] \<Rightarrow> 'b" (infixr "\<guillemotright>" 54) | |
| 54 | ||
| 37848 | 55 | syntax (latex output) | 
| 56 | "_thenM" :: "['a, 'b] \<Rightarrow> 'b" (infixr "\<then>" 54) | |
| 57 | ||
| 37790 | 58 | translations | 
| 59 | "_do_block (_do_cons (_do_then t) (_do_final e))" | |
| 37816 | 60 | == "CONST bind_do t (\<lambda>_. e)" | 
| 37790 | 61 | "_do_block (_do_cons (_do_bind p t) (_do_final e))" | 
| 37816 | 62 | == "CONST bind_do t (\<lambda>p. e)" | 
| 37790 | 63 | "_do_block (_do_cons (_do_let p t) bs)" | 
| 64 | == "let p = t in _do_block bs" | |
| 65 | "_do_block (_do_cons b (_do_cons c cs))" | |
| 66 | == "_do_block (_do_cons b (_do_final (_do_block (_do_cons c cs))))" | |
| 67 | "_do_cons (_do_let p t) (_do_final s)" | |
| 68 | == "_do_final (let p = t in s)" | |
| 69 | "_do_block (_do_final e)" => "e" | |
| 70 | "(m >> n)" => "(m >>= (\<lambda>_. n))" | |
| 71 | ||
| 37816 | 72 | setup {*
 | 
| 73 |   Adhoc_Overloading.add_overloaded @{const_name bind}
 | |
| 45964 | 74 |   #> Adhoc_Overloading.add_variant @{const_name bind} @{const_name Set.bind}
 | 
| 37816 | 75 |   #> Adhoc_Overloading.add_variant @{const_name bind} @{const_name Predicate.bind}
 | 
| 39151 | 76 |   #> Adhoc_Overloading.add_variant @{const_name bind} @{const_name Option.bind}
 | 
| 46143 | 77 |   #> Adhoc_Overloading.add_variant @{const_name bind} @{const_name List.bind}
 | 
| 37816 | 78 | *} | 
| 37790 | 79 | |
| 80 | end |