src/HOL/Map.thy
changeset 39992 f225a499a8e5
parent 39379 ab1b070aa412
child 41229 d797baa3d57c
--- a/src/HOL/Map.thy	Wed Oct 13 09:56:00 2010 +0200
+++ b/src/HOL/Map.thy	Sun Oct 10 22:50:25 2010 +0200
@@ -12,7 +12,6 @@
 begin
 
 types ('a,'b) "map" = "'a => 'b option" (infixr "~=>" 0)
-translations (type) "'a ~=> 'b" <= (type) "'a => 'b option"
 
 type_notation (xsymbols)
   "map" (infixr "\<rightharpoonup>" 0)