removed safe elim flag of trueElim and notFalseElim for testing.
--- a/src/HOL/HOL.thy Fri Mar 16 16:37:52 2007 +0100
+++ b/src/HOL/HOL.thy Fri Mar 16 16:40:49 2007 +0100
@@ -728,7 +728,7 @@
lemma TrueE: "True ==> P ==> P" .
lemma notFalseE: "~ False ==> P ==> P" .
-lemmas [Pure.elim!] = disjE iffE FalseE conjE exE TrueE notFalseE
+lemmas [Pure.elim!] = disjE iffE FalseE conjE exE
and [Pure.intro!] = iffI conjI impI TrueI notI allI refl
and [Pure.elim 2] = allE notE' impE'
and [Pure.intro] = exI disjI2 disjI1