src/HOL/Bali/Table.thy
changeset 24194 96013f81faef
parent 24038 18182c4aec9e
child 30235 58d147683393
--- a/src/HOL/Bali/Table.thy	Thu Aug 09 15:52:38 2007 +0200
+++ b/src/HOL/Bali/Table.thy	Thu Aug 09 15:52:42 2007 +0200
@@ -44,7 +44,7 @@
 translations
   "table_of" == "map_of"
   
-  (type)"'a \<rightharpoonup> 'b"       <= (type)"'a \<Rightarrow> 'b Option.option"
+  (type)"'a \<rightharpoonup> 'b"       <= (type)"'a \<Rightarrow> 'b Datatype.option"
   (type)"('a, 'b) table" <= (type)"'a \<rightharpoonup> 'b"
 
 (* ### To map *)