diff -r 2605ea41bbdd -r f14e41e9b08f Unused.thy --- a/Unused.thy Thu Jan 14 12:14:35 2010 +0100 +++ b/Unused.thy Thu Jan 14 12:17:39 2010 +0100 @@ -7,6 +7,30 @@ +(* Atomize infrastructure *) +(* FIXME/TODO: is this really needed? *) +(* +lemma atomize_eqv: + 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 +*) + ML {* fun dest_cbinop t =