--- a/Nominal/Nominal2_Atoms.thy Sun Mar 21 22:27:08 2010 +0100
+++ b/Nominal/Nominal2_Atoms.thy Mon Mar 22 09:16:25 2010 +0100
@@ -23,8 +23,6 @@
class at = at_base +
assumes sort_of_atom_eq [simp]: "sort_of (atom a) = sort_of (atom b)"
-instance at < at_base ..
-
lemma supp_at_base:
fixes a::"'a::at_base"
shows "supp a = {atom a}"
@@ -146,13 +144,12 @@
subsection {* Syntax for coercing at-elements to the atom-type *}
-(*
syntax
"_atom_constrain" :: "logic \<Rightarrow> type \<Rightarrow> logic" ("_:::_" [4, 0] 3)
translations
- "_atom_constrain a t" => "atom (_constrain a t)"
-*)
+ "_atom_constrain a t" => "CONST atom (_constrain a t)"
+
subsection {* A lemma for proving instances of class @{text at}. *}