src/HOL/Lex/Prefix.thy
author paulson
Thu, 18 Jan 1996 10:38:29 +0100
changeset 1444 23ceb1dc9755
parent 1344 f172a7f14e49
child 1476 608483c2122a
permissions -rw-r--r--
trivial updates

(*  Title: 	HOL/Lex/Prefix.thy
    ID:         $Id$
    Author: 	Tobias Nipkow
    Copyright   1995 TUM
*)

Prefix = List +

arities list :: (term)ord

defs
	prefix_def     "xs <= zs  ==  ? ys. zs = xs@ys"
end