src/HOL/Bali/Table.thy
changeset 35431 8758fe1fc9f8
parent 35417 47ee18b6ae32
child 37956 ee939247b2fb
--- a/src/HOL/Bali/Table.thy	Wed Mar 03 00:32:14 2010 +0100
+++ b/src/HOL/Bali/Table.thy	Wed Mar 03 00:33:02 2010 +0100
@@ -42,8 +42,7 @@
   where "table_of \<equiv> map_of"
 
 translations
-  (type)"'a \<rightharpoonup> 'b"       <= (type)"'a \<Rightarrow> 'b Datatype.option"
-  (type)"('a, 'b) table" <= (type)"'a \<rightharpoonup> 'b"
+  (type) "('a, 'b) table" <= (type) "'a \<rightharpoonup> 'b"
 
 (* ### To map *)
 lemma map_add_find_left[simp]: