src/HOL/UNITY/WFair.thy
changeset 35355 613e133966ea
parent 32693 6c6b1ba5e71e
child 35417 47ee18b6ae32
--- a/src/HOL/UNITY/WFair.thy	Wed Feb 24 22:04:10 2010 +0100
+++ b/src/HOL/UNITY/WFair.thy	Wed Feb 24 22:09:50 2010 +0100
@@ -69,8 +69,8 @@
      --{*predicate transformer: the largest set that leads to @{term B}*}
     "wlt F B == Union {A. F \<in> A leadsTo B}"
 
-syntax (xsymbols)
-  "op leadsTo" :: "['a set, 'a set] => 'a program set" (infixl "\<longmapsto>" 60)
+notation (xsymbols)
+  leadsTo  (infixl "\<longmapsto>" 60)
 
 
 subsection{*transient*}