changeset 524 | c7c6ba5ac043 |
parent 516 | bed81795848c |
child 526 | 7ba2fc25c6a3 |
--- a/FSet.thy Fri Dec 04 12:21:15 2009 +0100 +++ b/FSet.thy Fri Dec 04 13:58:23 2009 +0100 @@ -337,8 +337,6 @@ apply (tactic {* lift_tac_fset @{context} @{thm append_assoc} 1 *}) done -lemma cheat: "P" sorry - lemma "\<lbrakk>P EMPTY; \<And>a x. P x \<Longrightarrow> P (INSERT a x)\<rbrakk> \<Longrightarrow> P l" apply (tactic {* (ObjectLogic.full_atomize_tac THEN' gen_frees_tac @{context}) 1 *})