src/HOL/Extraction/Warshall.thy
changeset 16417 9bc16273c2d4
parent 13671 eec2582923f6
child 16761 99549528ce76
--- a/src/HOL/Extraction/Warshall.thy	Fri Jun 17 11:35:35 2005 +0200
+++ b/src/HOL/Extraction/Warshall.thy	Fri Jun 17 16:12:49 2005 +0200
@@ -5,7 +5,7 @@
 
 header {* Warshall's algorithm *}
 
-theory Warshall = Main:
+theory Warshall imports Main begin
 
 text {*
   Derivation of Warshall's algorithm using program extraction,