src/HOL/Bali/Table.thy
changeset 34939 44294cfecb1d
parent 30235 58d147683393
child 35355 613e133966ea
child 35416 d8d7d1b785af
--- a/src/HOL/Bali/Table.thy	Fri Jan 15 08:27:21 2010 +0100
+++ b/src/HOL/Bali/Table.thy	Sat Jan 16 17:15:27 2010 +0100
@@ -1,5 +1,4 @@
 (*  Title:      HOL/Bali/Table.thy
-    ID:         $Id$
     Author:     David von Oheimb
 *)
 header {* Abstract tables and their implementation as lists *}
@@ -41,9 +40,10 @@
 syntax
   table_of      :: "('a \<times> 'b) list \<Rightarrow> ('a, 'b) table"   --{* concrete table *}
   
+abbreviation
+  "table_of \<equiv> map_of"
+
 translations
-  "table_of" == "map_of"
-  
   (type)"'a \<rightharpoonup> 'b"       <= (type)"'a \<Rightarrow> 'b Datatype.option"
   (type)"('a, 'b) table" <= (type)"'a \<rightharpoonup> 'b"