src/HOL/Isar_examples/HoareEx.thy
changeset 16417 9bc16273c2d4
parent 15912 47aa1a8fcdc9
child 18193 54419506df9e
--- a/src/HOL/Isar_examples/HoareEx.thy	Fri Jun 17 11:35:35 2005 +0200
+++ b/src/HOL/Isar_examples/HoareEx.thy	Fri Jun 17 16:12:49 2005 +0200
@@ -1,7 +1,7 @@
 
 header {* Using Hoare Logic *}
 
-theory HoareEx = Hoare:
+theory HoareEx imports Hoare begin
 
 subsection {* State spaces *}