Prelude.thy
author urbanc
Thu, 28 Apr 2011 03:24:20 +0000
changeset 158 3c9129f49846
parent 35 d2ddce8b36fd
permissions -rw-r--r--
paper about formalising parsing; seems to have done what we would like to do....probably also appears at ITP'11

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