src/HOL/Bali/Decl.thy
changeset 12937 0c4fd7529467
parent 12925 99131847fb93
child 13601 fd3e3d6b37b2
--- a/src/HOL/Bali/Decl.thy	Mon Feb 25 20:46:09 2002 +0100
+++ b/src/HOL/Bali/Decl.thy	Mon Feb 25 20:48:14 2002 +0100
@@ -723,12 +723,12 @@
 qed
 
 lemma ws_interface_induct [consumes 2, case_names Step]:
- (assumes is_if_I: "is_iface G I" and 
+  assumes is_if_I: "is_iface G I" and 
                ws: "ws_prog G" and
           hyp_sub: "\<And>I i. \<lbrakk>iface G I = Some i; 
                             \<forall> J \<in> set (isuperIfs i).
                                  (I,J)\<in>subint1 G \<and> P J \<and> is_iface G J\<rbrakk> \<Longrightarrow> P I"
- ) "P I"
+  shows "P I"
 proof -
   from is_if_I ws 
   show "P I"