src/HOLCF/Fix.thy
changeset 18078 20e5a6440790
parent 18074 a92b7c5133de
child 18090 9d5cfd71f510
--- a/src/HOLCF/Fix.thy	Thu Nov 03 01:02:29 2005 +0100
+++ b/src/HOLCF/Fix.thy	Thu Nov 03 01:11:39 2005 +0100
@@ -33,13 +33,13 @@
 subsection {* Binder syntax for @{term fix} *}
 
 syntax
-  "_FIX" :: "[pttrn, 'a] => 'a" ("(3FIX _./ _)" [0, 10] 10)
+  "_FIX" :: "['a, 'a] \<Rightarrow> 'a" ("(3FIX _./ _)" [1000, 10] 10)
 
 syntax (xsymbols)
-  "_FIX" :: "[pttrn, 'a] => 'a" ("(3\<mu>_./ _)" [0, 10] 10)
+  "_FIX" :: "['a, 'a] \<Rightarrow> 'a" ("(3\<mu>_./ _)" [1000, 10] 10)
 
 translations
-  "FIX x. t" == "fix$(LAM x. t)"
+  "\<mu> x. t" == "fix\<cdot>(\<Lambda> x. t)"
 
 subsection {* Properties of @{term iterate} *}