author | haftmann |
Thu, 17 Jun 2010 15:59:48 +0200 | |
changeset 37450 | 45073611170a |
parent 36098 | 53992c639da5 |
child 37771 | 1bec64044b5e |
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" "ex/SatChecker" begin end