src/HOL/ex/LexProd.thy
changeset 3231 6d1768e1d9bc
parent 3230 3772723c5e41
child 3232 19a2b853ba7b
--- a/src/HOL/ex/LexProd.thy	Tue May 20 11:05:59 1997 +0200
+++ /dev/null	Thu Jan 01 00:00:00 1970 +0000
@@ -1,15 +0,0 @@
-(*  Title:      HOL/ex/lex-prod.thy
-    ID:         $Id$
-    Author:     Tobias Nipkow, TU Munich
-    Copyright   1993  TU Munich
-
-The lexicographic product of two relations.
-*)
-
-LexProd = WF + Prod +
-consts "**" :: "[('a*'a)set, ('b*'b)set] => (('a*'b)*('a*'b))set" (infixl 70)
-rules
-lex_prod_def "ra**rb == {p. ? a a' b b'. 
-        p = ((a,b),(a',b')) & ((a,a') : ra | a=a' & (b,b') : rb)}"
-end
-