src/HOL/Bali/Table.thy
changeset 12858 6214f03d6d27
parent 12857 a4386cc9b1c3
child 12925 99131847fb93
equal deleted inserted replaced
12857:a4386cc9b1c3 12858:6214f03d6d27
     1 (*  Title:      HOL/Bali/Table.thy
     1 (*  Title:      HOL/Bali/Table.thy
     2     ID:         $Id$
     2     ID:         $Id$
     3     Author:     David von Oheimb
     3     Author:     David von Oheimb
     4     Copyright   1997 Technische Universitaet Muenchen
     4     License:    GPL (GNU GENERAL PUBLIC LICENSE)
     5 *)
     5 *)
     6 header {* Abstract tables and their implementation as lists *}
     6 header {* Abstract tables and their implementation as lists *}
     7 
     7 
     8 theory Table = Basis:
     8 theory Table = Basis:
     9 
     9