# HG changeset patch # User berghofe # Date 1026399434 -7200 # Node ID 7d4441c8c46a1cbf9d1e731f7a45cbeedefd35ba # Parent 374d05460db4e206ed4e0c35f9f704fe6c556359 Added "using" to the beginning of original newman proof again, because it was lost during last update; renamed second version of newman to newman' (this allows for a comparison of the primitive proof objects, for example). diff -r 374d05460db4 -r 7d4441c8c46a src/HOL/Lambda/Commutation.thy --- a/src/HOL/Lambda/Commutation.thy Thu Jul 11 13:43:24 2002 +0200 +++ b/src/HOL/Lambda/Commutation.thy Thu Jul 11 16:57:14 2002 +0200 @@ -138,59 +138,60 @@ subsection {* Newman's lemma *} -(* Proof by Stefan Berghofer *) +text {* Proof by Stefan Berghofer *} 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 + shows "\b c. (a, b) \ R\<^sup>* \ (a, c) \ R\<^sup>* \ + \d. (b, d) \ R\<^sup>* \ (c, d) \ R\<^sup>*" + using wf +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 = b" - with xc have "(b, c) \ R\<^sup>*" by simp + assume "x = c" + with xb have "(c, b) \ 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[symmetric] 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 - note xy'[symmetric] - 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 + 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 -(* Partly automated by Tobias Nipkow. Takes 2 minutes (2002). *) +text {* + \medskip Alternative version. Partly automated by Tobias + Nipkow. Takes 2 minutes (2002). -text{* This is the maximal amount of automation possible at the moment. *} + This is the maximal amount of automation possible at the moment. +*} -theorem newman: +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>*"