author | berghofe |
Thu, 12 Jan 2012 00:13:37 +0100 | |
changeset 46191 | a88546428c2a |
parent 39307 | 8d42d668b5b0 |
child 50630 | 1ea90e8046dc |
permissions | -rw-r--r-- |
30694 | 1 |
(* Title: HOL/Imperative_HOL/Imperative_HOL_ex.thy |
31872 | 2 |
Author: John Matthews, Galois Connections; |
3 |
Alexander Krauss, Lukas Bulwahn & Florian Haftmann, TU Muenchen |
|
30694 | 4 |
*) |
5 |
||
31872 | 6 |
header {* Monadic imperative HOL with examples *} |
30694 | 7 |
|
8 |
theory Imperative_HOL_ex |
|
39307 | 9 |
imports Imperative_HOL Overview |
37771
1bec64044b5e
spelt out relational framework in a consistent way
haftmann
parents:
36098
diff
changeset
|
10 |
"ex/Imperative_Quicksort" "ex/Imperative_Reverse" "ex/Linked_Lists" "ex/SatChecker" |
30694 | 11 |
begin |
12 |
||
37831
fa3a2e35c4f1
repaired some implementations of imperative operations
haftmann
parents:
37829
diff
changeset
|
13 |
definition "everything = (Array.new, Array.of_list, Array.make, Array.len, Array.nth, |
37829 | 14 |
Array.upd, Array.map_entry, Array.swap, Array.freeze, |
37831
fa3a2e35c4f1
repaired some implementations of imperative operations
haftmann
parents:
37829
diff
changeset
|
15 |
ref, Ref.lookup, Ref.update, Ref.change)" |
37829 | 16 |
|
38058 | 17 |
export_code everything checking SML SML_imp OCaml? OCaml_imp? Haskell? Scala? Scala_imp? |
37826 | 18 |
|
30694 | 19 |
end |