proper support for "isabelle update -D DIR": avoid accidental exclusion of select_dirs (amending e5dafe9e120f);
(* Title: HOL/Eisbach/Eisbach_Old_Appl_Syntax.thy
Author: Makarius
*)
section \<open>Alternative Eisbach entry point for FOL, ZF etc.\<close>
theory Eisbach_Old_Appl_Syntax
imports Eisbach
begin
setup Pure_Thy.old_appl_syntax_setup
end