src/HOL/HoareParallel/RG_Hoare.thy
changeset 16417 9bc16273c2d4
parent 15236 f289e8ba2bb3
child 17528 2a602a8462d5
     1.1 --- a/src/HOL/HoareParallel/RG_Hoare.thy	Fri Jun 17 11:35:35 2005 +0200
     1.2 +++ b/src/HOL/HoareParallel/RG_Hoare.thy	Fri Jun 17 16:12:49 2005 +0200
     1.3 @@ -1,6 +1,6 @@
     1.4  header {* \section{The Proof System} *}
     1.5  
     1.6 -theory RG_Hoare = RG_Tran:
     1.7 +theory RG_Hoare imports RG_Tran begin
     1.8  
     1.9  subsection {* Proof System for Component Programs *}
    1.10