Nominal/ExPS6.thy
changeset 1604 5ab97f43ec24
parent 1600 e33e37fd4c7d
child 1655 9cec4269b7f9
--- a/Nominal/ExPS6.thy	Tue Mar 23 09:21:43 2010 +0100
+++ b/Nominal/ExPS6.thy	Tue Mar 23 09:34:32 2010 +0100
@@ -6,6 +6,9 @@
 
 atom_decl name
 
+(* The binding structure is too complicated, so we cannot show equivalence *)
+ML {* val _ = cheat_equivp := true *}
+
 ML {* val _ = recursive := false  *}
 nominal_datatype exp6 =
   EVar name
@@ -28,6 +31,7 @@
 thm exp6_pat6.perm
 thm exp6_pat6.induct
 thm exp6_pat6.distinct
+thm exp6_pat6.supp
 
 end