diff -r 6e0f56764ff8 -r dc95a56b1953 ProgTutorial/Package/Simple_Inductive_Package.thy
--- a/ProgTutorial/Package/Simple_Inductive_Package.thy	Wed Apr 29 00:36:14 2009 +0200
+++ b/ProgTutorial/Package/Simple_Inductive_Package.thy	Tue May 05 03:21:49 2009 +0200
@@ -44,7 +44,6 @@
 where
   accpartI': "\<And>x. (\<And>y. r y x \<Longrightarrow> accpart' y) \<Longrightarrow> accpart' x"
 
-
 context rel
 begin
   thm accpartI'