src/FOL/IFOL.thy
changeset 18481 b75ce99617c7
parent 17702 ea88ddeafabe
child 18523 9446cb8e1f65
--- a/src/FOL/IFOL.thy	Thu Dec 22 00:29:12 2005 +0100
+++ b/src/FOL/IFOL.thy	Thu Dec 22 00:29:14 2005 +0100
@@ -143,6 +143,15 @@
 
 use "IFOL_lemmas.ML"
 
+ML {*
+structure ProjectRule = ProjectRuleFun
+(struct
+  val conjunct1 = thm "conjunct1";
+  val conjunct2 = thm "conjunct2";
+  val mp = thm "mp";
+end)
+*}
+
 use "fologic.ML"
 use "hypsubstdata.ML"
 setup hypsubst_setup