src/HOLCF/Holcfb.thy
changeset 1168 74be52691d62
parent 243 c22b85994e17
child 1274 ea0668a1c0ba
--- a/src/HOLCF/Holcfb.thy	Thu Jun 29 16:16:24 1995 +0200
+++ b/src/HOLCF/Holcfb.thy	Thu Jun 29 16:28:40 1995 +0200
@@ -13,9 +13,9 @@
 
 theleast     :: "(nat=>bool)=>nat"
 
-rules
+defs
 
-theleast_def    "theleast(P) == (@z.(P(z) & (!n.P(n)-->z<=n)))"
+theleast_def    "theleast P == (@z.(P z & (!n.P n --> z<=n)))"
 
 end