author | lcp |
Tue, 25 Apr 1995 11:14:03 +0200 | |
changeset 1072 | 0140ff702b23 |
parent 972 | e61b058d58d2 |
child 1151 | c820b3cc3df0 |
permissions | -rw-r--r-- |
969 | 1 |
(* Title: HOL/ex/lex-prod.thy |
2 |
ID: $Id$ |
|
3 |
Author: Tobias Nipkow, TU Munich |
|
4 |
Copyright 1993 TU Munich |
|
5 |
||
6 |
The lexicographic product of two relations. |
|
7 |
*) |
|
8 |
||
9 |
LexProd = WF + Prod + |
|
10 |
consts "**" :: "[('a*'a)set, ('b*'b)set] => (('a*'b)*('a*'b))set" (infixl 70) |
|
11 |
rules |
|
12 |
lex_prod_def "ra**rb == {p. ? a a' b b'. \ |
|
972
e61b058d58d2
changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents:
969
diff
changeset
|
13 |
\ p = ((a,b),(a',b')) & ((a,a') : ra | a=a' & (b,b') : rb)}" |
969 | 14 |
end |
15 |