| author | wenzelm |
| Wed, 15 Aug 2001 22:20:30 +0200 | |
| changeset 11501 | 3b6415035d1a |
| parent 11319 | 8b84ee2cc79c |
| child 12593 | cd35fe5947d4 |
| permissions | -rw-r--r-- |
(* Title: Confluence.thy ID: $Id$ Author: Ole Rasmussen Copyright 1995 University of Cambridge Logic Image: ZF *) Confluence = Reduction+ consts confluence :: i=>o strip :: o defs confluence_def "confluence(R) == \\<forall>x y. <x,y>:R --> (\\<forall>z.<x,z>:R --> (\\<exists>u.<y,u>:R & <z,u>:R))" strip_def "strip == \\<forall>x y. (x ===> y) --> (\\<forall>z.(x =1=> z) --> (\\<exists>u.(y =1=> u) & (z===>u)))" end