Automatic computation of application preservation and manually finished "alpha.induct". Slow...
authorCezary Kaliszyk <kaliszyk@in.tum.de>
Sat, 31 Oct 2009 11:20:55 +0100
changeset 253 e169a99c6ada
parent 252 e30997c88050
child 255 264c7b9d19f4
Automatic computation of application preservation and manually finished "alpha.induct". Slow...
FSet.thy
LamEx.thy
QuotMain.thy
QuotScript.thy
--- a/FSet.thy	Fri Oct 30 19:03:53 2009 +0100
+++ b/FSet.thy	Sat Oct 31 11:20:55 2009 +0100
@@ -356,18 +356,10 @@
 
 ML {* val abs = findabs rty (prop_of (atomize_thm @{thm list.induct})) *}
 ML {* val aps = findaps rty (prop_of (atomize_thm @{thm list.induct})) *}
-
-ML {* val simp_lam_prs_thms = map (make_simp_lam_prs_thm @{context} quot) abs *}
-ML {* val ind_r_l = repeat_eqsubst_thm @{context} simp_lam_prs_thms ind_r_t *}
-lemma app_prs_for_induct: "(ABS_fset ---> id) f (REP_fset T1) = f T1"
-  apply (simp add: fun_map.simps QUOT_TYPE_I_fset.thm10)
-done
-
-ML {* val ind_r_l1 = eqsubst_thm @{context} @{thms app_prs_for_induct} ind_r_l *}
-ML {* val ind_r_l2 = eqsubst_thm @{context} @{thms app_prs_for_induct} ind_r_l1 *}
-ML {* val ind_r_l3 = eqsubst_thm @{context} @{thms app_prs_for_induct} ind_r_l2 *}
-ML {* val ind_r_l4 = eqsubst_thm @{context} @{thms app_prs_for_induct} ind_r_l3 *}
-ML {* val ind_r_a = simp_allex_prs @{context} quot ind_r_l4 *}
+ML {* val simp_app_prs_thms = map (make_simp_prs_thm @{context} quot @{thm APP_PRS}) aps *}
+ML {* val simp_lam_prs_thms = map (make_simp_prs_thm @{context} quot @{thm LAMBDA_PRS}) abs *}
+ML {* val ind_r_l = repeat_eqsubst_thm @{context} (simp_app_prs_thms @ simp_lam_prs_thms) ind_r_t *}
+ML {* val ind_r_a = simp_allex_prs @{context} quot ind_r_l *}
 ML {* val thm = @{thm FORALL_PRS[OF FUN_QUOTIENT[OF QUOTIENT_fset IDENTITY_QUOTIENT], symmetric]} *}
 ML {* val ind_r_a1 = eqsubst_thm @{context} [thm] ind_r_a *}
 ML {* val defs_sym = add_lower_defs @{context} defs *}
--- a/LamEx.thy	Fri Oct 30 19:03:53 2009 +0100
+++ b/LamEx.thy	Sat Oct 31 11:20:55 2009 +0100
@@ -196,6 +196,7 @@
 
 thm rlam.inject
 thm pi_var
+ 
 
 lemma var_inject:
   shows "(Var a = Var b) = (a = b)"
@@ -221,19 +222,54 @@
 
 
 
-ML {* val t_a = atomize_thm @{thm alpha.cases} *}
+ML {* val t_a = atomize_thm @{thm alpha.induct} *}
+(* prove {* build_regularize_goal t_a rty rel @{context}  *}
+ML_prf {*  fun tac ctxt =
+     (FIRST' [
+      rtac rel_refl,
+      atac,
+      rtac @{thm universal_twice},
+      (rtac @{thm impI} THEN' atac),
+      rtac @{thm implication_twice},
+      EqSubst.eqsubst_tac ctxt [0]
+        [(@{thm equiv_res_forall} OF [rel_eqv]),
+         (@{thm equiv_res_exists} OF [rel_eqv])],
+      (rtac @{thm impI} THEN' (asm_full_simp_tac (Simplifier.context ctxt HOL_ss)) THEN' rtac rel_refl),
+      (rtac @{thm RIGHT_RES_FORALL_REGULAR})
+     ]);
+ *}
+  apply (tactic {* tac @{context} 1 *}) *)
 ML {* val t_r = regularize t_a rty rel rel_eqv rel_refl @{context} *}
 ML {* val t_t = repabs @{context} t_r consts rty qty quot rel_refl trans2 rsp_thms *}
-ML {* val abs = findabs rty (prop_of t_a); *}
-ML {* val simp_lam_prs_thms = map (make_simp_lam_prs_thm @{context} quot) abs *}
-ML {* val t_l = repeat_eqsubst_thm @{context} simp_lam_prs_thms t_t *}
+
+ML {* val abs = findabs rty (prop_of (atomize_thm @{thm alpha.induct})) *}
+ML {* val aps = findaps rty (prop_of (atomize_thm @{thm alpha.induct})) *}
+ML {* val aps = @{typ "LamEx.rlam \<Rightarrow> bool"} :: aps; *}
+ML {* val simp_app_prs_thms = map (make_simp_prs_thm @{context} quot @{thm APP_PRS}) aps *}
+ML {* val simp_lam_prs_thms = map (make_simp_prs_thm @{context} quot @{thm LAMBDA_PRS}) abs *}
+ML {* val t_l = repeat_eqsubst_thm @{context} (simp_app_prs_thms @ simp_lam_prs_thms) t_t *}
 ML {* val t_a = simp_allex_prs @{context} quot t_l *}
+ML {* val thm = 
+  @{thm FORALL_PRS[OF FUN_QUOTIENT[OF QUOTIENT_lam FUN_QUOTIENT[OF QUOTIENT_lam IDENTITY_QUOTIENT]], symmetric]} *}
+ML {* val t_a1 = eqsubst_thm @{context} [thm] t_a *}
 ML {* val defs_sym = add_lower_defs @{context} defs; *}
-ML {* val t_d = repeat_eqsubst_thm @{context} defs_sym t_a *}
+ML {* val t_d = repeat_eqsubst_thm @{context} defs_sym t_a1 *}
 ML {* val t_r = MetaSimplifier.rewrite_rule [reps_same] t_d *}
-ML {* ObjectLogic.rulify t_r *}
+ML {* val t_r1 = repeat_eqsubst_thm @{context} @{thms fun_map.simps} t_r *}
+ML {* val t_r2 = repeat_eqsubst_thm @{context} @{thms QUOT_TYPE_I_lam.thm10} t_r1 *}
+ML {* val t_r3 = repeat_eqsubst_thm @{context} @{thms id_apply} t_r2 *}
+
+ML {* val alpha_induct = ObjectLogic.rulify t_r3 *}
 
+local_setup {*
+  Quotient.note (@{binding "alpha_induct"}, alpha_induct) #> snd
+*}
 
+lemma
+  assumes a: "(a::lam) = b"
+  shows "False"
+  using a
+  apply (rule alpha_induct)
 
 fun
   option_map::"('a \<Rightarrow> 'b) \<Rightarrow> ('a noption) \<Rightarrow> ('b noption)"
--- a/QuotMain.thy	Fri Oct 30 19:03:53 2009 +0100
+++ b/QuotMain.thy	Sat Oct 31 11:20:55 2009 +0100
@@ -535,10 +535,11 @@
       rtac rel_refl,
       atac,
       rtac @{thm universal_twice},
+      (rtac @{thm impI} THEN' atac),
       rtac @{thm implication_twice},
-      (fn i => CHANGED (asm_full_simp_tac ((Simplifier.context ctxt HOL_ss) addsimps
+      EqSubst.eqsubst_tac ctxt [0]
         [(@{thm equiv_res_forall} OF [rel_eqv]),
-         (@{thm equiv_res_exists} OF [rel_eqv])]) i)),
+         (@{thm equiv_res_exists} OF [rel_eqv])],
       (rtac @{thm impI} THEN' (asm_full_simp_tac (Simplifier.context ctxt HOL_ss)) THEN' rtac rel_refl),
       (rtac @{thm RIGHT_RES_FORALL_REGULAR})
      ]);
@@ -848,26 +849,25 @@
       Abs(_, T, b) =>
         findaps_all rty (subst_bound ((Free ("x", T)), b))
     | (f $ a) => (findaps_all rty f @ findaps_all rty a)
-    | Free (_, (T as (Type (_, (_ :: _))))) => (if needs_lift rty T then [T] else [])
+    | Free (_, (T as (Type ("fun", (_ :: _))))) => (if needs_lift rty T then [T] else [])
     | _ => [];
   fun findaps rty tm = distinct (op =) (findaps_all rty tm)
 *}
 
 ML {*
-fun make_simp_lam_prs_thm lthy quot_thm typ =
+fun make_simp_prs_thm lthy quot_thm thm typ =
   let
     val (_, [lty, rty]) = dest_Type typ;
     val thy = ProofContext.theory_of lthy;
     val (lcty, rcty) = (ctyp_of thy lty, ctyp_of thy rty)
     val inst = [SOME lcty, NONE, SOME rcty];
-    val lpi = Drule.instantiate' inst [] @{thm LAMBDA_PRS};
+    val lpi = Drule.instantiate' inst [] thm;
     val tac =
-      (compose_tac (false, @{thm LAMBDA_PRS}, 2)) THEN_ALL_NEW
+      (compose_tac (false, lpi, 2)) THEN_ALL_NEW
       (quotient_tac quot_thm);
     val t = Goal.prove lthy [] [] (concl_of lpi) (fn _ => tac 1);
-    val ts = @{thm HOL.sym} OF [t]
   in
-    MetaSimplifier.rewrite_rule [@{thm eq_reflection} OF @{thms id_apply}] ts
+    MetaSimplifier.rewrite_rule [@{thm eq_reflection} OF @{thms id_apply}] t
   end
 *}
 
@@ -929,8 +929,10 @@
   val t_r = regularize t_a rty rel rel_eqv rel_refl lthy;
   val t_t = repabs lthy t_r consts rty qty quot rel_refl trans2 rsp_thms;
   val abs = findabs rty (prop_of t_a);
-  val simp_lam_prs_thms = map (make_simp_lam_prs_thm lthy quot) abs;
-  val t_l = repeat_eqsubst_thm lthy simp_lam_prs_thms t_t;
+  val aps = findaps rty (prop_of t_a);
+  val app_prs_thms = map (make_simp_prs_thm lthy quot @{thm APP_PRS}) aps;
+  val lam_prs_thms = map (make_simp_prs_thm lthy quot @{thm LAMBDA_PRS}) abs;
+  val t_l = repeat_eqsubst_thm lthy (lam_prs_thms @ app_prs_thms) t_t;
   val t_a = simp_allex_prs lthy quot t_l;
   val defs_sym = add_lower_defs lthy defs;
   val t_d = repeat_eqsubst_thm lthy defs_sym t_a;
--- a/QuotScript.thy	Fri Oct 30 19:03:53 2009 +0100
+++ b/QuotScript.thy	Sat Oct 31 11:20:55 2009 +0100
@@ -274,7 +274,7 @@
 lemma LAMBDA_PRS:
   assumes q1: "QUOTIENT R1 Abs1 Rep1"
   and     q2: "QUOTIENT R2 Abs2 Rep2"
-  shows "(\<lambda>x. f x) = (Rep1 ---> Abs2) (\<lambda>x. Rep2 (f (Abs1 x)))"
+  shows "(Rep1 ---> Abs2) (\<lambda>x. Rep2 (f (Abs1 x))) = (\<lambda>x. f x)"
 unfolding expand_fun_eq
 using QUOTIENT_ABS_REP[OF q1] QUOTIENT_ABS_REP[OF q2]
 by simp
@@ -284,7 +284,16 @@
   and     q2: "QUOTIENT R2 Abs2 Rep2"
   shows "(\<lambda>x. f x) = (Rep1 ---> Abs2) (\<lambda>x. (Abs1 ---> Rep2) f x)"
 unfolding expand_fun_eq
-by (subst LAMBDA_PRS[OF q1 q2]) (simp)
+using QUOTIENT_ABS_REP[OF q1] QUOTIENT_ABS_REP[OF q2]
+by (simp)
+
+lemma APP_PRS:
+  assumes q1: "QUOTIENT R1 abs1 rep1"
+  and     q2: "QUOTIENT R2 abs2 rep2"
+  shows "abs2 ((abs1 ---> rep2) f (rep1 x)) = f x"
+unfolding expand_fun_eq
+using QUOTIENT_ABS_REP[OF q1] QUOTIENT_ABS_REP[OF q2]
+by simp
 
 (* Ask Peter: assumption q1 and q2 not used and lemma is the 'identity' *)
 lemma LAMBDA_RSP: