ProgTutorial/Package/Simple_Inductive_Package.thy
changeset 244 dc95a56b1953
parent 189 069d525f8f1d
child 316 74f0a06f751f
--- 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'