src/HOL/Map.thy
changeset 25483 65de74f62874
parent 24331 76f7a8c6e842
child 25490 e8ab1c42c14f
--- a/src/HOL/Map.thy	Wed Nov 28 09:01:37 2007 +0100
+++ b/src/HOL/Map.thy	Wed Nov 28 09:01:39 2007 +0100
@@ -12,11 +12,11 @@
 imports List
 begin
 
-types ('a,'b) "~=>" = "'a => 'b option"  (infixr 0)
+types ('a,'b) map = "'a => 'b option"  (infixr "~=>" 0)
 translations (type) "a ~=> b " <= (type) "a => b option"
 
 syntax (xsymbols)
-  "~=>" :: "[type, type] => type"  (infixr "\<rightharpoonup>" 0)
+  map :: "type \<Rightarrow> type \<Rightarrow> type"  (infixr "\<rightharpoonup>" 0)
 
 abbreviation
   empty :: "'a ~=> 'b" where