diff -r 790d1863be28 -r 824f8390aaa2 src/HOL/MetisExamples/TransClosure.thy --- a/src/HOL/MetisExamples/TransClosure.thy Tue Oct 14 15:45:46 2008 +0200 +++ b/src/HOL/MetisExamples/TransClosure.thy Tue Oct 14 16:01:36 2008 +0200 @@ -22,7 +22,7 @@ consts f:: "addr \ val" -ML {*AtpThread.problem_name := "TransClosure__test"*} +ML {*AtpWrapper.problem_name := "TransClosure__test"*} lemma "\ f c = Intg x; \ y. f b = Intg y \ y \ x; (a,b) \ R\<^sup>*; (b,c) \ R\<^sup>* \ \ \ c. (b,c) \ R \ (a,c) \ R\<^sup>*" by (metis Transitive_Closure.rtrancl_into_rtrancl converse_rtranclE trancl_reflcl) @@ -51,7 +51,7 @@ by (metis 10 3) qed -ML {*AtpThread.problem_name := "TransClosure__test_simpler"*} +ML {*AtpWrapper.problem_name := "TransClosure__test_simpler"*} lemma "\ f c = Intg x; \ y. f b = Intg y \ y \ x; (a,b) \ R\<^sup>*; (b,c) \ R\<^sup>* \ \ \ c. (b,c) \ R \ (a,c) \ R\<^sup>*" apply (erule_tac x="b" in converse_rtranclE)