src/HOL/Imperative_HOL/Imperative_HOL_ex.thy
changeset 37771 1bec64044b5e
parent 36098 53992c639da5
child 37826 4c0a5e35931a
--- a/src/HOL/Imperative_HOL/Imperative_HOL_ex.thy	Mon Jul 12 11:39:27 2010 +0200
+++ b/src/HOL/Imperative_HOL/Imperative_HOL_ex.thy	Mon Jul 12 16:05:08 2010 +0200
@@ -6,8 +6,8 @@
 header {* Monadic imperative HOL with examples *}
 
 theory Imperative_HOL_ex
-imports Imperative_HOL "ex/Imperative_Quicksort" "ex/Imperative_Reverse" "ex/Linked_Lists"
-  "ex/SatChecker"
+imports Imperative_HOL
+  "ex/Imperative_Quicksort" "ex/Imperative_Reverse" "ex/Linked_Lists" "ex/SatChecker"
 begin
 
 end