disabled spurious invocation of (interactive) sledgehammer;
authorwenzelm
Wed, 28 Apr 2010 19:43:45 +0200
changeset 36501 6c7ba330ab42
parent 36500 620f899158d4
child 36502 586af36cf3cc
child 36512 875218f3f97c
disabled spurious invocation of (interactive) sledgehammer;
src/HOL/Metis_Examples/TransClosure.thy
--- a/src/HOL/Metis_Examples/TransClosure.thy	Wed Apr 28 17:29:58 2010 +0200
+++ b/src/HOL/Metis_Examples/TransClosure.thy	Wed Apr 28 19:43:45 2010 +0200
@@ -23,7 +23,7 @@
 
 lemma "\<lbrakk>f c = Intg x; \<forall>y. f b = Intg y \<longrightarrow> y \<noteq> x; (a, b) \<in> R\<^sup>*; (b, c) \<in> R\<^sup>*\<rbrakk>
        \<Longrightarrow> \<exists>c. (b, c) \<in> R \<and> (a, c) \<in> R\<^sup>*"
-sledgehammer
+(* sledgehammer *)
 proof -
   assume A1: "f c = Intg x"
   assume A2: "\<forall>y. f b = Intg y \<longrightarrow> y \<noteq> x"