src/HOL/Import/ImportRecorder.thy
author wenzelm
Thu, 14 Aug 2008 16:52:46 +0200
changeset 27865 27a8ad9612a3
parent 20594 b80c4a5cd018
permissions -rw-r--r--
moved basic thm operations from structure PureThy to Thm (cf. more_thm.ML);

theory ImportRecorder imports Main 
uses  "seq.ML" "scan.ML" "mono_seq.ML" "mono_scan.ML" "lazy_seq.ML" "xml.ML" "xmlconv.ML" "importrecorder.ML"
begin
end