diff -r 4e5bd3883429 -r 557302525778 src/HOL/BNF/Examples/TreeFsetI.thy --- a/src/HOL/BNF/Examples/TreeFsetI.thy Wed Sep 26 10:00:59 2012 +0200 +++ b/src/HOL/BNF/Examples/TreeFsetI.thy Wed Sep 26 10:00:59 2012 +0200 @@ -50,7 +50,7 @@ apply (simp add: pre_treeFsetI_rel_def prod_rel_def fset_rel_def) done -lemmas treeFsetI_coind = mp[OF treeFsetI.dtor_rel_coinduct] +lemmas treeFsetI_coind = mp[OF treeFsetI.dtor_coinduct] lemma "tmap (f o g) x = tmap f (tmap g x)" by (intro treeFsetI_coind[where P="%x1 x2. \x. x1 = tmap (f o g) x \ x2 = tmap f (tmap g x)"])