tuned whitespace
authortraytel
Sun, 08 Sep 2013 12:26:07 +0200
changeset 53470 fe80dd7cd543
parent 53469 3356a148b783
child 53471 66df4b76e58f
tuned whitespace
src/HOL/BNF/Examples/TreeFI.thy
--- a/src/HOL/BNF/Examples/TreeFI.thy	Sun Sep 08 12:26:05 2013 +0200
+++ b/src/HOL/BNF/Examples/TreeFI.thy	Sun Sep 08 12:26:07 2013 +0200
@@ -27,12 +27,12 @@
   unfolding trev_def by simp
 
 lemma treeFI_coinduct:
-assumes *: "phi x y"
-and step: "\<And>a b. phi a b \<Longrightarrow>
-   lab a = lab b \<and>
-   lengthh (sub a) = lengthh (sub b) \<and>
-   (\<forall>i < lengthh (sub a). phi (nthh (sub a) i) (nthh (sub b) i))"
-shows "x = y"
+  assumes *: "phi x y"
+  and step: "\<And>a b. phi a b \<Longrightarrow>
+     lab a = lab b \<and>
+     lengthh (sub a) = lengthh (sub b) \<and>
+     (\<forall>i < lengthh (sub a). phi (nthh (sub a) i) (nthh (sub b) i))"
+  shows "x = y"
 using * proof (coinduct rule: treeFI.coinduct)
   fix t1 t2 assume "phi t1 t2" note * = step[OF this] and ** = conjunct2[OF *]
   from conjunct1[OF **] conjunct2[OF **] have "relF phi (sub t1) (sub t2)"