diff -r ce5f78f0eac5 -r 2a19e0a37131 Quot/QuotMain.thy --- a/Quot/QuotMain.thy Thu Jan 14 10:06:29 2010 +0100 +++ b/Quot/QuotMain.thy Thu Jan 14 10:47:19 2010 +0100 @@ -148,30 +148,6 @@ use "quotient_tacs.ML" -(* Atomize infrastructure *) -(* FIXME/TODO: is this really needed? *) -(* -lemma atomize_eqv[atomize]: - shows "(Trueprop A \ Trueprop B) \ (A \ B)" -proof - assume "A \ B" - then show "Trueprop A \ Trueprop B" by unfold -next - assume *: "Trueprop A \ Trueprop B" - have "A = B" - proof (cases A) - case True - have "A" by fact - then show "A = B" using * by simp - next - case False - have "\A" by fact - then show "A = B" using * by auto - qed - then show "A \ B" by (rule eq_reflection) -qed -*) - section {* Methods / Interface *} ML {*