src/HOLCF/Tr1.thy
changeset 1168 74be52691d62
parent 625 119391dd1d59
child 1274 ea0668a1c0ba
--- a/src/HOLCF/Tr1.thy	Thu Jun 29 16:16:24 1995 +0200
+++ b/src/HOLCF/Tr1.thy	Thu Jun 29 16:28:40 1995 +0200
@@ -31,22 +31,14 @@
 
 rules
 
-  abs_tr_iso	"abs_tr[rep_tr[u]] = u"
-  rep_tr_iso	"rep_tr[abs_tr[x]] = x"
+  abs_tr_iso	"abs_tr`(rep_tr`u) = u"
+  rep_tr_iso	"rep_tr`(abs_tr`x) = x"
 
-  TT_def	"TT == abs_tr[sinl[one]]"
-  FF_def	"FF == abs_tr[sinr[one]]"
-
-  tr_when_def "tr_when == (LAM e1 e2 t.when[LAM x.e1][LAM y.e2][rep_tr[t]])"
-
-end
+defs
 
-
-
-
-
+  TT_def	"TT == abs_tr`(sinl`one)"
+  FF_def	"FF == abs_tr`(sinr`one)"
 
-
-
-
-
+  tr_when_def "tr_when == 
+	(LAM e1 e2 t. sswhen`(LAM x.e1)`(LAM y.e2)`(rep_tr`t))"
+end