| author | wenzelm | 
| Mon, 20 Oct 2014 23:17:28 +0200 | |
| changeset 58728 | 42398b610f86 | 
| parent 53109 | 186535065f5c | 
| child 58889 | 5b7a9633cfa8 | 
| permissions | -rw-r--r-- | 
| 29822 | 1 | (* Title: HOL/Imperative_HOL/Imperative_HOL.thy | 
| 26170 | 2 | Author: John Matthews, Galois Connections; Alexander Krauss, Lukas Bulwahn & Florian Haftmann, TU Muenchen | 
| 3 | *) | |
| 4 | ||
| 5 | header {* Entry point into monadic imperative HOL *}
 | |
| 6 | ||
| 7 | theory Imperative_HOL | |
| 53109 
186535065f5c
renamed theory Mrec to Legacy_Mrec, no longer included by default
 krauss parents: 
37776diff
changeset | 8 | imports Array Ref | 
| 26170 | 9 | begin | 
| 10 | ||
| 11 | end |