# HG changeset patch # User blanchet # Date 1347617367 -7200 # Node ID d9800bc28427cbbcd4be60c9f3632d5ea514089f # Parent df359ce891ac5170b23e3fc7e4f1987234fca45f compile diff -r df359ce891ac -r d9800bc28427 src/HOL/Codatatype/Examples/Stream.thy --- a/src/HOL/Codatatype/Examples/Stream.thy Fri Sep 14 12:09:27 2012 +0200 +++ b/src/HOL/Codatatype/Examples/Stream.thy Fri Sep 14 12:09:27 2012 +0200 @@ -133,27 +133,27 @@ definition ns :: "nat \ nat stream" where [simp]: "ns n = scalar n ones" lemma "ones \ ones = twos" -by (intro stream_coind[where phi="%x1 x2. \x. x1 = ones \ ones \ x2 = twos"]) +by (intro stream_coind[where P="%x1 x2. \x. x1 = ones \ ones \ x2 = twos"]) auto lemma "n \ twos = ns (2 * n)" -by (intro stream_coind[where phi="%x1 x2. \n. x1 = n \ twos \ x2 = ns (2 * n)"]) +by (intro stream_coind[where P="%x1 x2. \n. x1 = n \ twos \ x2 = ns (2 * n)"]) force+ lemma prod_scalar: "(n * m) \ xs = n \ m \ xs" -by (intro stream_coind[where phi="%x1 x2. \n m xs. x1 = (n * m) \ xs \ x2 = n \ m \ xs"]) +by (intro stream_coind[where P="%x1 x2. \n m xs. x1 = (n * m) \ xs \ x2 = n \ m \ xs"]) force+ lemma scalar_plus: "n \ (xs \ ys) = n \ xs \ n \ ys" -by (intro stream_coind[where phi="%x1 x2. \n xs ys. x1 = n \ (xs \ ys) \ x2 = n \ xs \ n \ ys"]) +by (intro stream_coind[where P="%x1 x2. \n xs ys. x1 = n \ (xs \ ys) \ x2 = n \ xs \ n \ ys"]) (force simp: add_mult_distrib2)+ lemma plus_comm: "xs \ ys = ys \ xs" -by (intro stream_coind[where phi="%x1 x2. \xs ys. x1 = xs \ ys \ x2 = ys \ xs"]) +by (intro stream_coind[where P="%x1 x2. \xs ys. x1 = xs \ ys \ x2 = ys \ xs"]) force+ lemma plus_assoc: "(xs \ ys) \ zs = xs \ ys \ zs" -by (intro stream_coind[where phi="%x1 x2. \xs ys zs. x1 = (xs \ ys) \ zs \ x2 = xs \ ys \ zs"]) +by (intro stream_coind[where P="%x1 x2. \xs ys zs. x1 = (xs \ ys) \ zs \ x2 = xs \ ys \ zs"]) force+ end diff -r df359ce891ac -r d9800bc28427 src/HOL/Codatatype/Examples/TreeFsetI.thy --- a/src/HOL/Codatatype/Examples/TreeFsetI.thy Fri Sep 14 12:09:27 2012 +0200 +++ b/src/HOL/Codatatype/Examples/TreeFsetI.thy Fri Sep 14 12:09:27 2012 +0200 @@ -52,7 +52,7 @@ lemmas treeFsetI_coind = mp[OF treeFsetI.pred_coinduct] lemma "tmap (f o g) x = tmap f (tmap g x)" -by (intro treeFsetI_coind[where phi="%x1 x2. \x. x1 = tmap (f o g) x \ x2 = 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)"]) force+ end