Attic/Prelude.thy
author urbanc
Wed, 29 Aug 2012 13:05:25 +0000
changeset 366 827e487b9e92
parent 170 b1258b7d2789
permissions -rw-r--r--
added slides for talk at Imperial
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
35
d2ddce8b36fd made the theory work under both Isabelle 2009 and 2011
urbanc
parents:
diff changeset
     1
theory Prelude
d2ddce8b36fd made the theory work under both Isabelle 2009 and 2011
urbanc
parents:
diff changeset
     2
imports Main
d2ddce8b36fd made the theory work under both Isabelle 2009 and 2011
urbanc
parents:
diff changeset
     3
begin
d2ddce8b36fd made the theory work under both Isabelle 2009 and 2011
urbanc
parents:
diff changeset
     4
d2ddce8b36fd made the theory work under both Isabelle 2009 and 2011
urbanc
parents:
diff changeset
     5
(*
d2ddce8b36fd made the theory work under both Isabelle 2009 and 2011
urbanc
parents:
diff changeset
     6
To make the theory work under Isabelle 2009 and 2011
d2ddce8b36fd made the theory work under both Isabelle 2009 and 2011
urbanc
parents:
diff changeset
     7
d2ddce8b36fd made the theory work under both Isabelle 2009 and 2011
urbanc
parents:
diff changeset
     8
Isabelle 2009: set_ext
d2ddce8b36fd made the theory work under both Isabelle 2009 and 2011
urbanc
parents:
diff changeset
     9
Isabelle 2011: set_eqI
d2ddce8b36fd made the theory work under both Isabelle 2009 and 2011
urbanc
parents:
diff changeset
    10
d2ddce8b36fd made the theory work under both Isabelle 2009 and 2011
urbanc
parents:
diff changeset
    11
*)
d2ddce8b36fd made the theory work under both Isabelle 2009 and 2011
urbanc
parents:
diff changeset
    12
d2ddce8b36fd made the theory work under both Isabelle 2009 and 2011
urbanc
parents:
diff changeset
    13
d2ddce8b36fd made the theory work under both Isabelle 2009 and 2011
urbanc
parents:
diff changeset
    14
lemma set_eq_intro:
d2ddce8b36fd made the theory work under both Isabelle 2009 and 2011
urbanc
parents:
diff changeset
    15
  "(\<And>x. (x \<in> A) = (x \<in> B)) \<Longrightarrow> A = B"
d2ddce8b36fd made the theory work under both Isabelle 2009 and 2011
urbanc
parents:
diff changeset
    16
by blast
d2ddce8b36fd made the theory work under both Isabelle 2009 and 2011
urbanc
parents:
diff changeset
    17
d2ddce8b36fd made the theory work under both Isabelle 2009 and 2011
urbanc
parents:
diff changeset
    18
d2ddce8b36fd made the theory work under both Isabelle 2009 and 2011
urbanc
parents:
diff changeset
    19
end