uses ("LCF_lemmas.ML");
authorwenzelm
Sat, 03 Sep 2005 17:56:48 +0200
changeset 17249 e89fbfd778c1
parent 17248 81bf91654e73
child 17250 158ef530c153
uses ("LCF_lemmas.ML");
src/LCF/LCF.thy
--- a/src/LCF/LCF.thy	Sat Sep 03 17:54:10 2005 +0200
+++ b/src/LCF/LCF.thy	Sat Sep 03 17:56:48 2005 +0200
@@ -8,7 +8,7 @@
 
 theory LCF
 imports FOL
-uses ("pair.ML") ("fix.ML")
+uses ("LCF_lemmas.ML") ("pair.ML") ("fix.ML")
 begin
 
 text {* This theory is based on Lawrence Paulson's book Logic and Computation. *}