src/HOL/BNF/Examples/TreeFI.thy
changeset 49588 9b72d207617b
parent 49510 ba50d204095e
child 49594 55e798614c45
--- a/src/HOL/BNF/Examples/TreeFI.thy	Wed Sep 26 10:00:59 2012 +0200
+++ b/src/HOL/BNF/Examples/TreeFI.thy	Wed Sep 26 10:00:59 2012 +0200
@@ -52,7 +52,7 @@
    lengthh (sub a) = lengthh (sub b) \<and>
    (\<forall>i < lengthh (sub a). phi (nthh (sub a) i) (nthh (sub b) i))"
 shows "x = y"
-proof (rule mp[OF treeFI.dtor_coinduct, of phi, OF _ *])
+proof (rule mp[OF treeFI.dtor_map_coinduct, of phi, OF _ *])
   fix a b :: "'a treeFI"
   let ?zs = "zipp (sub a) (sub b)"
   let ?z = "(lab a, ?zs)"