diff -r 6061ae1f90f2 -r 9bc16273c2d4 src/HOL/IMP/Machines.thy --- 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 \ (R O R^*)" by(fast intro:rtrancl.intros elim:rtranclE)