changeset 1150 | 66512c9e6bd6 |
parent 442 | 13ac1fd0a14d |
child 1168 | 74be52691d62 |
--- a/src/HOLCF/Cfun3.thy Wed Jun 21 15:01:07 1995 +0200 +++ b/src/HOLCF/Cfun3.thy Wed Jun 21 15:14:58 1995 +0200 @@ -19,9 +19,9 @@ inst_cfun_pcpo "(UU::'a->'b) = UU_cfun" -Istrictify_def "Istrictify(f,x) == (@z.\ -\ ( x=UU --> z = UU)\ -\ & (~x=UU --> z = f[x]))" +Istrictify_def "Istrictify(f,x) == (@z. + ( x=UU --> z = UU) + & (~x=UU --> z = f[x]))" strictify_def "strictify == (LAM f x.Istrictify(f,x))"