| author | wenzelm |
| Thu, 18 Mar 2010 23:00:18 +0100 | |
| changeset 35836 | 9380fab5f4f7 |
| parent 34051 | 1a82e2e29d67 |
| child 36098 | 53992c639da5 |
| permissions | -rw-r--r-- |
(* Title: HOL/Imperative_HOL/Imperative_HOL_ex.thy Author: John Matthews, Galois Connections; Alexander Krauss, Lukas Bulwahn & Florian Haftmann, TU Muenchen *) header {* Monadic imperative HOL with examples *} theory Imperative_HOL_ex imports Imperative_HOL "ex/Imperative_Quicksort" "ex/Imperative_Reverse" "ex/Linked_Lists" begin end