src/HOL/IMP/Machines.thy
changeset 16417 9bc16273c2d4
parent 14565 c6dc17aab88a
child 18372 2bffdf62fe7f
--- a/src/HOL/IMP/Machines.thy	Fri Jun 17 11:35:35 2005 +0200
+++ b/src/HOL/IMP/Machines.thy	Fri Jun 17 16:12:49 2005 +0200
@@ -1,4 +1,4 @@
-theory Machines = Natural:
+theory Machines imports Natural begin
 
 lemma rtrancl_eq: "R^* = Id \<union> (R O R^*)"
 by(fast intro:rtrancl.intros elim:rtranclE)