changeset 1168 | 74be52691d62 |
parent 1150 | 66512c9e6bd6 |
child 1479 | 21eb5e156d91 |
--- a/src/HOLCF/Cfun3.thy Thu Jun 29 16:16:24 1995 +0200 +++ b/src/HOLCF/Cfun3.thy Thu Jun 29 16:28:40 1995 +0200 @@ -19,13 +19,11 @@ inst_cfun_pcpo "(UU::'a->'b) = UU_cfun" -Istrictify_def "Istrictify(f,x) == (@z. - ( x=UU --> z = UU) - & (~x=UU --> z = f[x]))" +defs -strictify_def "strictify == (LAM f x.Istrictify(f,x))" +Istrictify_def "Istrictify f x == if x=UU then UU else f`x" + +strictify_def "strictify == (LAM f x.Istrictify f x)" end - -