src/HOL/Hoare/ExamplesAbort.thy
changeset 16417 9bc16273c2d4
parent 13875 12997e3ddd8d
child 16733 236dfafbeb63
--- a/src/HOL/Hoare/ExamplesAbort.thy	Fri Jun 17 11:35:35 2005 +0200
+++ b/src/HOL/Hoare/ExamplesAbort.thy	Fri Jun 17 16:12:49 2005 +0200
@@ -6,7 +6,7 @@
 Some small examples for programs that may abort.
 *)
 
-theory ExamplesAbort = HoareAbort:
+theory ExamplesAbort imports HoareAbort begin
 
 lemma "VARS x y z::nat
  {y = z & z \<noteq> 0} z \<noteq> 0 \<rightarrow> x := y div z {x = 1}"