src/HOL/Imperative_HOL/Imperative_HOL.thy
author berghofe
Fri, 27 Nov 2009 16:26:23 +0100
changeset 33935 b94b4587106a
parent 29822 c45845743f04
child 37772 026ed2fc15d4
permissions -rw-r--r--
Removed eq_to_mono2, added not_mono.
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
29822
c45845743f04 authentic syntax for List.nth
haftmann
parents: 29399
diff changeset
     1
(*  Title:      HOL/Imperative_HOL/Imperative_HOL.thy
26170
66e6b967ccf1 added theories for imperative HOL
haftmann
parents:
diff changeset
     2
    Author:     John Matthews, Galois Connections; Alexander Krauss, Lukas Bulwahn & Florian Haftmann, TU Muenchen
66e6b967ccf1 added theories for imperative HOL
haftmann
parents:
diff changeset
     3
*)
66e6b967ccf1 added theories for imperative HOL
haftmann
parents:
diff changeset
     4
66e6b967ccf1 added theories for imperative HOL
haftmann
parents:
diff changeset
     5
header {* Entry point into monadic imperative HOL *}
66e6b967ccf1 added theories for imperative HOL
haftmann
parents:
diff changeset
     6
66e6b967ccf1 added theories for imperative HOL
haftmann
parents:
diff changeset
     7
theory Imperative_HOL
27656
d4f6e64ee7cc added verification framework for the HeapMonad and quicksort as example for this framework
bulwahn
parents: 26170
diff changeset
     8
imports Array Ref Relational
26170
66e6b967ccf1 added theories for imperative HOL
haftmann
parents:
diff changeset
     9
begin
66e6b967ccf1 added theories for imperative HOL
haftmann
parents:
diff changeset
    10
66e6b967ccf1 added theories for imperative HOL
haftmann
parents:
diff changeset
    11
end