do not restore old files on startup, which is potentially slow due to automatic rechecking;
attempt to enable thick caret for improved visibility;
(* Title: HOL/ex/Interpretation_with_Defs.thy
Author: Florian Haftmann, TU Muenchen
*)
header {* Interpretation accompanied with mixin definitions. EXPERIMENTAL. *}
theory Interpretation_with_Defs
imports Pure
uses "~~/src/Tools/interpretation_with_defs.ML"
begin
end