src/ZF/ex/Commutation.thy
author wenzelm
Sat, 20 Oct 2001 20:20:41 +0200
changeset 11852 a528a716a312
parent 11316 b4e71bd751e4
child 12867 5c900a821a7c
permissions -rw-r--r--
added TextIO.stdErr;

(*  Title:      HOL/Lambda/Commutation.thy
    ID:         $Id$
    Author:     Tobias Nipkow & Sidi Ould Ehmety
    Copyright   1995  TU Muenchen

Commutation theory for proving the Church Rosser theorem
	ported from Isabelle/HOL  by Sidi Ould Ehmety
*)

Commutation = Main +    

constdefs
  square  :: [i, i, i, i] => o
   "square(r,s,t,u) ==
   (\\<forall>a b. <a,b>:r --> (\\<forall>c. <a, c>:s
                          --> (\\<exists>x. <b,x>:t & <c,x>:u)))"

   commute :: [i, i] => o       
   "commute(r,s) == square(r,s,s,r)"

  diamond :: i=>o
  "diamond(r)   == commute(r, r)"

  strip :: i=>o  
  "strip(r) == commute(r^*, r)"

  Church_Rosser :: i => o     
  "Church_Rosser(r) == (\\<forall>x y. <x,y>: (r Un converse(r))^* -->
			(\\<exists>z. <x,z>:r^* & <y,z>:r^*))"
  confluent :: i=>o    
  "confluent(r) == diamond(r^*)"
end