author | wenzelm |
Wed, 02 Aug 2000 19:40:14 +0200 | |
changeset 9502 | 50ec59aff389 |
parent 9156 | b9fe44ad3381 |
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 |
||
8523 | 7 |
Prefix = Main + |
1344 | 8 |
|
9156 | 9 |
instance list :: (term)ord |
1344 | 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 |