diff -r f04b33ce250f -r a4dc62a46ee4 ex/LexProd.thy
--- a/ex/LexProd.thy Tue Oct 24 14:59:17 1995 +0100
+++ /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 = <,> & ( : ra | a=a' & : rb)}"
-end
-