Attic/Prelude.thy
author Christian Urban <christian dot urban at kcl dot ac dot uk>
Thu, 11 Jul 2013 12:07:11 +0100
changeset 383 c8cb6914f4c8
parent 170 b1258b7d2789
permissions -rw-r--r--
some more polishing

theory Prelude
imports Main
begin

(*
To make the theory work under Isabelle 2009 and 2011

Isabelle 2009: set_ext
Isabelle 2011: set_eqI

*)


lemma set_eq_intro:
  "(\<And>x. (x \<in> A) = (x \<in> B)) \<Longrightarrow> A = B"
by blast


end