--- a/Nominal/Parser.thy Fri Mar 19 12:28:35 2010 +0100
+++ b/Nominal/Parser.thy Fri Mar 19 14:54:30 2010 +0100
@@ -271,9 +271,9 @@
ML {* val cheat_equivp = Unsynchronized.ref true *}
-(* Fixes for these 2 are known *)
-ML {* val cheat_fv_eqvt = Unsynchronized.ref true *} (* The tactic works, building the goal needs fixing *)
-ML {* val cheat_alpha_eqvt = Unsynchronized.ref true *} (* The tactic works, building the goal needs fixing *)
+(* These 2 are not needed any more *)
+ML {* val cheat_fv_eqvt = Unsynchronized.ref false *}
+ML {* val cheat_alpha_eqvt = Unsynchronized.ref false *}
ML {*
@@ -408,8 +408,8 @@
val (_, lthy20) = Local_Theory.note ((Binding.empty,
[Attrib.internal (fn _ => Nominal_ThmDecls.eqvt_add)]), q_eqvt) lthy19;
val _ = tracing "Finite Support";
- val supports = map (prove_supports lthy20 q_perm) consts handle _ => []
- val fin_supp = HOLogic.conj_elims (prove_fs lthy20 q_induct supports q_tys) handle _ => []
+ val supports = map (prove_supports lthy20 q_perm) consts;
+ val fin_supp = HOLogic.conj_elims (prove_fs lthy20 q_induct supports q_tys);
val thy3 = Local_Theory.exit_global lthy20;
val lthy21 = Theory_Target.instantiation (qty_full_names, [], @{sort fs}) thy3;
fun tac _ = Class.intro_classes_tac [] THEN (ALLGOALS (resolve_tac fin_supp))