src/FOL/IFOL.thy
changeset 12019 abe9b7c6016e
parent 11976 075df6e46cef
child 12114 a8e860c86252
--- a/src/FOL/IFOL.thy	Fri Nov 02 17:55:24 2001 +0100
+++ b/src/FOL/IFOL.thy	Fri Nov 02 22:01:07 2001 +0100
@@ -188,12 +188,11 @@
   Note that this list of rules is in reverse order of priorities.
 *}
 
-lemmas trans_rules [trans] =
+lemmas basic_trans_rules [trans] =
   forw_subst
   back_subst
   rev_mp
   mp
-  transitive
   trans
 
 lemmas [Pure.elim] = sym