| author | wenzelm |
| Mon, 12 Jul 1999 22:25:39 +0200 | |
| changeset 6980 | bb526ba7ba5f |
| parent 6675 | 63e53327f5e5 |
| child 8523 | 7ffc94f2f42d |
| permissions | -rw-r--r-- |
| 1476 | 1 |
(* Title: HOL/Lex/Prefix.thy |
| 1344 | 2 |
ID: $Id$ |
| 1476 | 3 |
Author: Tobias Nipkow |
| 1344 | 4 |
Copyright 1995 TUM |
5 |
*) |
|
6 |
||
7 |
Prefix = List + |
|
8 |
||
9 |
arities list :: (term)ord |
|
10 |
||
11 |
defs |
|
|
6675
63e53327f5e5
changes to show that Lists are partially ordered by the prefix relation
paulson
parents:
1476
diff
changeset
|
12 |
prefix_def "xs <= zs == ? ys. zs = xs@ys" |
|
63e53327f5e5
changes to show that Lists are partially ordered by the prefix relation
paulson
parents:
1476
diff
changeset
|
13 |
|
|
63e53327f5e5
changes to show that Lists are partially ordered by the prefix relation
paulson
parents:
1476
diff
changeset
|
14 |
strict_prefix_def "xs < zs == xs <= zs & xs ~= (zs::'a list)" |
|
63e53327f5e5
changes to show that Lists are partially ordered by the prefix relation
paulson
parents:
1476
diff
changeset
|
15 |
|
| 1344 | 16 |
end |