# HG changeset patch # User berghofe # Date 1019219584 -7200 # Node ID c8c28a1dc787ee68426850511c993af39aa35bdd # Parent 56b21879c603cec76379ae3a502a984b21cbc46d Added proof of Newman's lemma. diff -r 56b21879c603 -r c8c28a1dc787 src/HOL/Lambda/Commutation.thy --- a/src/HOL/Lambda/Commutation.thy Tue Apr 16 12:23:49 2002 +0200 +++ b/src/HOL/Lambda/Commutation.thy Fri Apr 19 14:33:04 2002 +0200 @@ -135,4 +135,53 @@ apply (blast del: rtrancl_refl intro: rtrancl_trans) done + +subsection {* Newman's lemma *} + +theorem newman: + assumes wf: "wf (R\)" + and lc: "\a b c. (a, b) \ R \ (a, c) \ R \ + \d. (b, d) \ R\<^sup>* \ (c, d) \ R\<^sup>*" + shows "(a, b) \ R\<^sup>* \ (a, c) \ R\<^sup>* \ + \d. (b, d) \ R\<^sup>* \ (c, d) \ R\<^sup>*" (is "PROP ?conf b c") +proof - + from wf show "\b c. PROP ?conf b c" + proof induct + case (less x b c) + have xc: "(x, c) \ R\<^sup>*" . + have xb: "(x, b) \ R\<^sup>*" . thus ?case + proof (rule converse_rtranclE) + assume "x = b" + with xc have "(b, c) \ R\<^sup>*" by simp + thus ?thesis by rules + next + fix y + assume xy: "(x, y) \ R" + assume yb: "(y, b) \ R\<^sup>*" + from xc show ?thesis + proof (rule converse_rtranclE) + assume "x = c" + with xb have "(c, b) \ R\<^sup>*" by simp + thus ?thesis by rules + next + fix y' + assume y'c: "(y', c) \ R\<^sup>*" + assume xy': "(x, y') \ R" + with xy have "\u. (y, u) \ R\<^sup>* \ (y', u) \ R\<^sup>*" by (rule lc) + then obtain u where yu: "(y, u) \ R\<^sup>*" and y'u: "(y', u) \ R\<^sup>*" by rules + from xy have "(y, x) \ R\" .. + from this and yb yu have "\d. (b, d) \ R\<^sup>* \ (u, d) \ R\<^sup>*" by (rule less) + then obtain v where bv: "(b, v) \ R\<^sup>*" and uv: "(u, v) \ R\<^sup>*" by rules + from xy' have "(y', x) \ R\" .. + moreover from y'u and uv have "(y', v) \ R\<^sup>*" by (rule rtrancl_trans) + moreover note y'c + ultimately have "\d. (v, d) \ R\<^sup>* \ (c, d) \ R\<^sup>*" by (rule less) + then obtain w where vw: "(v, w) \ R\<^sup>*" and cw: "(c, w) \ R\<^sup>*" by rules + from bv vw have "(b, w) \ R\<^sup>*" by (rule rtrancl_trans) + with cw show ?thesis by rules + qed + qed + qed +qed + end