added definition of string prefix and string subtraction
theory Preludeimports Mainbegin(*To make the theory work under Isabelle 2009 and 2011Isabelle 2009: set_extIsabelle 2011: set_eqI*)lemma set_eq_intro: "(\<And>x. (x \<in> A) = (x \<in> B)) \<Longrightarrow> A = B"by blastend