added warning and automatic deactivation of HTML generation if we cannot write
.theory_list.txt;
fixed bug which occured when index_path's value is "/"
(* Title: Sigs.thy
ID: $Id$
Author: Markus Wenzel, TU Muenchen
*)
Sigs = HOL +
axclass
inv < term
axclass
one < term
consts
"inv" :: "'a::inv => 'a"
"1" :: "'a::one" ("1")
end