src/HOLCF/Dnat.thy
changeset 1168 74be52691d62
parent 1150 66512c9e6bd6
--- a/src/HOLCF/Dnat.thy	Thu Jun 29 16:16:24 1995 +0200
+++ b/src/HOLCF/Dnat.thy	Thu Jun 29 16:28:40 1995 +0200
@@ -61,38 +61,40 @@
 (* dnat_abs is an isomorphism with inverse dnat_rep                        *)
 (* identity is the least endomorphism on dnat                              *)
 
-dnat_abs_iso	"dnat_rep[dnat_abs[x]] = x"
-dnat_rep_iso	"dnat_abs[dnat_rep[x]] = x"
+dnat_abs_iso	"dnat_rep`(dnat_abs`x) = x"
+dnat_rep_iso	"dnat_abs`(dnat_rep`x) = x"
 dnat_copy_def	"dnat_copy == (LAM f. dnat_abs oo 
-		 (when[sinl][sinr oo f]) oo dnat_rep )"
-dnat_reach	"(fix[dnat_copy])[x]=x"
+		 (sswhen`sinl`(sinr oo f)) oo dnat_rep )"
+dnat_reach	"(fix`dnat_copy)`x=x"
 
+
+defs
 (* ----------------------------------------------------------------------- *)
 (* properties of additional constants                                      *)
 (* ----------------------------------------------------------------------- *)
 (* constructors                                                            *)
 
-dzero_def	"dzero == dnat_abs[sinl[one]]"
-dsucc_def	"dsucc == (LAM n. dnat_abs[sinr[n]])"
+dzero_def	"dzero == dnat_abs`(sinl`one)"
+dsucc_def	"dsucc == (LAM n. dnat_abs`(sinr`n))"
 
 (* ----------------------------------------------------------------------- *)
 (* discriminator functional                                                *)
 
-dnat_when_def	"dnat_when == (LAM f1 f2 n.when[LAM x.f1][f2][dnat_rep[n]])"
+dnat_when_def	"dnat_when == (LAM f1 f2 n.sswhen`(LAM x.f1)`f2`(dnat_rep`n))"
 
 
 (* ----------------------------------------------------------------------- *)
 (* discriminators and selectors                                            *)
 
-is_dzero_def	"is_dzero == dnat_when[TT][LAM x.FF]"
-is_dsucc_def	"is_dsucc == dnat_when[FF][LAM x.TT]"
-dpred_def	"dpred == dnat_when[UU][LAM x.x]"
+is_dzero_def	"is_dzero == dnat_when`TT`(LAM x.FF)"
+is_dsucc_def	"is_dsucc == dnat_when`FF`(LAM x.TT)"
+dpred_def	"dpred == dnat_when`UU`(LAM x.x)"
 
 
 (* ----------------------------------------------------------------------- *)
 (* the taker for dnats                                                   *)
 
-dnat_take_def "dnat_take == (%n.iterate(n,dnat_copy,UU))"
+dnat_take_def "dnat_take == (%n.iterate n dnat_copy UU)"
 
 (* ----------------------------------------------------------------------- *)
 (* definition of bisimulation is determined by domain equation             *)
@@ -100,13 +102,9 @@
 
 dnat_bisim_def "dnat_bisim ==
 (%R.!s1 s2.
- 	R(s1,s2) -->
+ 	R s1 s2 -->
   ((s1=UU & s2=UU) |(s1=dzero & s2=dzero) |
-  (? s11 s21. s11~=UU & s21~=UU & s1=dsucc[s11] &
-		 s2 = dsucc[s21] & R(s11,s21))))"
+  (? s11 s21. s11~=UU & s21~=UU & s1=dsucc`s11 &
+		 s2 = dsucc`s21 & R s11 s21)))"
 
 end
-
-
-
-