src/HOL/Import/ImportRecorder.thy
author blanchet
Mon, 06 Jun 2011 20:36:35 +0200
changeset 43188 0c36ae874fcc
parent 20594 b80c4a5cd018
permissions -rw-r--r--
fixed detection of Skolem constants in type construction detection code

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