src/HOL/HOL.thy
changeset 48195 3127f9ce52fb
parent 48073 1b609a7837ef
child 48776 37cd53e69840
--- a/src/HOL/HOL.thy	Thu Jul 05 16:53:29 2012 +0200
+++ b/src/HOL/HOL.thy	Thu Jul 05 16:58:03 2012 +0200
@@ -404,14 +404,6 @@
 lemma eq_neq_eq_imp_neq: "[| x = a ; a ~= b; b = y |] ==> x ~= y"
   by (erule subst, erule ssubst, assumption)
 
-(*still used in HOLCF*)
-lemma rev_contrapos:
-  assumes pq: "P ==> Q"
-      and nq: "~Q"
-  shows "~P"
-apply (rule nq [THEN contrapos_nn])
-apply (erule pq)
-done
 
 subsubsection {*Existential quantifier*}