removed obsolete rev_contrapos (cf. 1d195de59497);
authorwenzelm
Thu, 05 Jul 2012 16:58:03 +0200
changeset 48195 3127f9ce52fb
parent 48194 1440a3103af0
child 48196 b7313810b6e6
removed obsolete rev_contrapos (cf. 1d195de59497);
src/HOL/HOL.thy
--- 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*}