removed obsolete/unused pred_congs;
authorwenzelm
Wed, 11 Jun 2008 18:01:11 +0200
changeset 27151 bd387c1a0536
parent 27150 a42aef558ce3
child 27152 192954a9a549
removed obsolete/unused pred_congs;
src/FOL/IFOL.thy
--- a/src/FOL/IFOL.thy	Wed Jun 11 15:41:57 2008 +0200
+++ b/src/FOL/IFOL.thy	Wed Jun 11 18:01:11 2008 +0200
@@ -518,16 +518,6 @@
   apply assumption
   done
 
-(*special cases for free variables P, Q, R, S -- up to 3 arguments*)
-
-ML {*
-bind_thms ("pred_congs",
-  List.concat (map (fn c => 
-               map (fn th => read_instantiate [("P",c)] th)
-                   [@{thm pred1_cong}, @{thm pred2_cong}, @{thm pred3_cong}])
-               (explode"PQRS")))
-*}
-
 (*special case for the equality predicate!*)
 lemma eq_cong: "[| a = a'; b = b' |] ==> a = b <-> a' = b'"
   apply (erule (1) pred2_cong)