made the subtyping work again
authorChristian Urban <urbanc@in.tum.de>
Tue, 10 May 2011 17:10:22 +0100
changeset 2782 2cb34b1e7e19
parent 2781 542ff50555f5
child 2783 8412c7e503d4
made the subtyping work again
Nominal/Atoms.thy
--- a/Nominal/Atoms.thy	Tue May 10 07:47:06 2011 +0100
+++ b/Nominal/Atoms.thy	Tue May 10 17:10:22 2011 +0100
@@ -3,9 +3,9 @@
 
     Instantiations of concrete atoms 
 *)
+
 theory Atoms
 imports Nominal2_Base
-uses "~~/src/Tools/subtyping.ML"
 begin
 
 
@@ -225,12 +225,11 @@
 
 declare [[coercion "atom::var2\<Rightarrow>atom"]]
 
-(*
 lemma
   fixes a::"var1" and b::"var2"
   shows "a \<sharp> t \<and> b \<sharp> t"
 oops
-*)
+
 
 (* does not yet work: it needs image as
    coercion map *)