src/HOL/Bali/Table.thy
changeset 13337 f75dfc606ac7
parent 12925 99131847fb93
child 13585 db4005b40cc6
--- a/src/HOL/Bali/Table.thy	Wed Jul 10 14:51:18 2002 +0200
+++ b/src/HOL/Bali/Table.thy	Wed Jul 10 15:07:02 2002 +0200
@@ -41,7 +41,7 @@
 
 syntax
   table_of      :: "('a \<times> 'b) list \<Rightarrow> ('a, 'b) table"    (* concrete table *)
-
+  
 translations
   "table_of" == "map_of"