src/HOL/Nominal/nominal_inductive2.ML
author wenzelm
Fri, 08 Dec 2023 16:01:42 +0100
changeset 79209 fe24edf8acda
parent 78812 d769a183d51d
child 80634 a90ab1ea6458
permissions -rw-r--r--
tuned;
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
     1
(*  Title:      HOL/Nominal/nominal_inductive2.ML
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
     2
    Author:     Stefan Berghofer, TU Muenchen
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
     3
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
     4
Infrastructure for proving equivariance and strong induction theorems
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
     5
for inductive predicates involving nominal datatypes.
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
     6
Experimental version that allows to avoid lists of atoms.
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
     7
*)
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
     8
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
     9
signature NOMINAL_INDUCTIVE2 =
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
    10
sig
38715
6513ea67d95d renamed Simplifier.simproc(_i) to Simplifier.simproc_global(_i) to emphasize that this is not the real thing;
wenzelm
parents: 38558
diff changeset
    11
  val prove_strong_ind: string -> string option -> (string * string list) list ->
6513ea67d95d renamed Simplifier.simproc(_i) to Simplifier.simproc_global(_i) to emphasize that this is not the real thing;
wenzelm
parents: 38558
diff changeset
    12
    local_theory -> Proof.state
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
    13
end
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
    14
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
    15
structure NominalInductive2 : NOMINAL_INDUCTIVE2 =
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
    16
struct
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
    17
59940
087d81f5213e local setup of induction tools, with restricted access to auxiliary consts;
wenzelm
parents: 59936
diff changeset
    18
val inductive_forall_def = @{thm HOL.induct_forall_def};
33772
b6a1feca2ac2 use of thm-antiquotation
Christian Urban <urbanc@in.tum.de>
parents: 33671
diff changeset
    19
val inductive_atomize = @{thms induct_atomize};
b6a1feca2ac2 use of thm-antiquotation
Christian Urban <urbanc@in.tum.de>
parents: 33671
diff changeset
    20
val inductive_rulify = @{thms induct_rulify};
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
    21
41228
e1fce873b814 renamed structure MetaSimplifier to raw_Simplifer, to emphasize its meaning;
wenzelm
parents: 39557
diff changeset
    22
fun rulify_term thy = Raw_Simplifier.rewrite_term thy inductive_rulify [];
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
    23
51717
9e7d1c139569 simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents: 50771
diff changeset
    24
fun atomize_conv ctxt =
41228
e1fce873b814 renamed structure MetaSimplifier to raw_Simplifer, to emphasize its meaning;
wenzelm
parents: 39557
diff changeset
    25
  Raw_Simplifier.rewrite_cterm (true, false, false) (K (K NONE))
51717
9e7d1c139569 simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents: 50771
diff changeset
    26
    (put_simpset HOL_basic_ss ctxt addsimps inductive_atomize);
9e7d1c139569 simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents: 50771
diff changeset
    27
fun atomize_intr ctxt = Conv.fconv_rule (Conv.prems_conv ~1 (atomize_conv ctxt));
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
    28
fun atomize_induct ctxt = Conv.fconv_rule (Conv.prems_conv ~1
74524
8ee3d5d3c1bf more accurate treatment of context, notably for nested Goal.proof / SUBPROOF;
wenzelm
parents: 74523
diff changeset
    29
  (Conv.params_conv ~1 (Conv.prems_conv ~1 o atomize_conv) ctxt));
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
    30
51717
9e7d1c139569 simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents: 50771
diff changeset
    31
fun fresh_postprocess ctxt =
9e7d1c139569 simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents: 50771
diff changeset
    32
  Simplifier.full_simplify (put_simpset HOL_basic_ss ctxt addsimps
30108
bd78f08b0ba1 Added postprocessing rules for fresh_star.
berghofe
parents: 30087
diff changeset
    33
    [@{thm fresh_star_set_eq}, @{thm fresh_star_Un_elim},
bd78f08b0ba1 Added postprocessing rules for fresh_star.
berghofe
parents: 30087
diff changeset
    34
     @{thm fresh_star_insert_elim}, @{thm fresh_star_empty_elim}]);
bd78f08b0ba1 Added postprocessing rules for fresh_star.
berghofe
parents: 30087
diff changeset
    35
44929
haftmann
parents: 44868
diff changeset
    36
fun preds_of ps t = inter (op = o apsnd dest_Free) ps (Term.add_frees t []);
30087
a780642a9c9c nominal_inductive and equivariance now work on local_theory.
berghofe
parents: 29585
diff changeset
    37
44689
f247fc952f31 tuned specifications
haftmann
parents: 44241
diff changeset
    38
val perm_bool = mk_meta_eq @{thm perm_bool_def};
39159
0dec18004e75 more antiquotations;
wenzelm
parents: 38795
diff changeset
    39
val perm_boolI = @{thm perm_boolI};
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
    40
val (_, [perm_boolI_pi, _]) = Drule.strip_comb (snd (Thm.dest_comb
59582
0fbed69ff081 tuned signature -- prefer qualified names;
wenzelm
parents: 59498
diff changeset
    41
  (Drule.strip_imp_concl (Thm.cprop_of perm_boolI))));
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
    42
60787
12cd198f07af updated to infer_instantiate;
wenzelm
parents: 60754
diff changeset
    43
fun mk_perm_bool ctxt pi th =
12cd198f07af updated to infer_instantiate;
wenzelm
parents: 60754
diff changeset
    44
  th RS infer_instantiate ctxt [(#1 (dest_Var (Thm.term_of perm_boolI_pi)), pi)] perm_boolI;
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
    45
60359
cb8828b859a1 clarified context;
wenzelm
parents: 59940
diff changeset
    46
fun mk_perm_bool_simproc names =
78812
d769a183d51d simprocs may be distinguished via 'identifier': only works for ML antiquotation (see also 13252110a6fe);
wenzelm
parents: 78806
diff changeset
    47
  Simplifier.make_simproc \<^context>
d769a183d51d simprocs may be distinguished via 'identifier': only works for ML antiquotation (see also 13252110a6fe);
wenzelm
parents: 78806
diff changeset
    48
   {name = "perm_bool",
d769a183d51d simprocs may be distinguished via 'identifier': only works for ML antiquotation (see also 13252110a6fe);
wenzelm
parents: 78806
diff changeset
    49
    lhss = [\<^term>\<open>perm pi x\<close>],
61144
5e94dfead1c2 simplified simproc programming interfaces;
wenzelm
parents: 60801
diff changeset
    50
    proc = fn _ => fn _ => fn ct =>
5e94dfead1c2 simplified simproc programming interfaces;
wenzelm
parents: 60801
diff changeset
    51
      (case Thm.term_of ct of
69597
ff784d5a5bfb isabelle update -u control_cartouches;
wenzelm
parents: 67522
diff changeset
    52
        Const (\<^const_name>\<open>Nominal.perm\<close>, _) $ _ $ t =>
67405
e9ab4ad7bd15 uniform use of Standard ML op-infix -- eliminated warnings;
wenzelm
parents: 67399
diff changeset
    53
          if member (op =) names (the_default "" (try (head_of #> dest_Const #> fst) t))
61144
5e94dfead1c2 simplified simproc programming interfaces;
wenzelm
parents: 60801
diff changeset
    54
          then SOME perm_bool else NONE
78812
d769a183d51d simprocs may be distinguished via 'identifier': only works for ML antiquotation (see also 13252110a6fe);
wenzelm
parents: 78806
diff changeset
    55
       | _ => NONE),
d769a183d51d simprocs may be distinguished via 'identifier': only works for ML antiquotation (see also 13252110a6fe);
wenzelm
parents: 78806
diff changeset
    56
    identifier = []};
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
    57
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
    58
fun transp ([] :: _) = []
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
    59
  | transp xs = map hd xs :: transp (map tl xs);
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
    60
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
    61
fun add_binders thy i (t as (_ $ _)) bs = (case strip_comb t of
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
    62
      (Const (s, T), ts) => (case strip_type T of
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
    63
        (Ts, Type (tname, _)) =>
31938
f193d95b4632 nominal.ML is nominal_datatype.ML
haftmann
parents: 31723
diff changeset
    64
          (case NominalDatatype.get_nominal_datatype thy tname of
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
    65
             NONE => fold (add_binders thy i) ts bs
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
    66
           | SOME {descr, index, ...} => (case AList.lookup op =
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
    67
                 (#3 (the (AList.lookup op = descr index))) s of
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
    68
               NONE => fold (add_binders thy i) ts bs
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
    69
             | SOME cargs => fst (fold (fn (xs, x) => fn (bs', cargs') =>
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
    70
                 let val (cargs1, (u, _) :: cargs2) = chop (length xs) cargs'
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
    71
                 in (add_binders thy i u
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
    72
                   (fold (fn (u, T) =>
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
    73
                      if exists (fn j => j < i) (loose_bnos u) then I
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
    74
                      else AList.map_default op = (T, [])
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
    75
                        (insert op aconv (incr_boundvars (~i) u)))
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
    76
                          cargs1 bs'), cargs2)
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
    77
                 end) cargs (bs, ts ~~ Ts))))
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
    78
      | _ => fold (add_binders thy i) ts bs)
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
    79
    | (u, ts) => add_binders thy i u (fold (add_binders thy i) ts bs))
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
    80
  | add_binders thy i (Abs (_, _, t)) bs = add_binders thy (i + 1) t bs
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
    81
  | add_binders thy i _ bs = bs;
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
    82
69597
ff784d5a5bfb isabelle update -u control_cartouches;
wenzelm
parents: 67522
diff changeset
    83
fun split_conj f names (Const (\<^const_name>\<open>HOL.conj\<close>, _) $ p $ q) _ = (case head_of p of
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
    84
      Const (name, _) =>
36692
54b64d4ad524 farewell to old-style mem infixes -- type inference in situations with mem_int and mem_string should provide enough information to resolve the type of (op =)
haftmann
parents: 36428
diff changeset
    85
        if member (op =) names name then SOME (f p q) else NONE
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
    86
    | _ => NONE)
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
    87
  | split_conj _ _ _ _ = NONE;
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
    88
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
    89
fun strip_all [] t = t
69597
ff784d5a5bfb isabelle update -u control_cartouches;
wenzelm
parents: 67522
diff changeset
    90
  | strip_all (_ :: xs) (Const (\<^const_name>\<open>All\<close>, _) $ Abs (s, T, t)) = strip_all xs t;
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
    91
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
    92
(*********************************************************************)
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
    93
(* maps  R ... & (ALL pi_1 ... pi_n z. P z (pi_1 o ... o pi_n o t))  *)
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
    94
(* or    ALL pi_1 ... pi_n z. P z (pi_1 o ... o pi_n o t)            *)
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
    95
(* to    R ... & id (ALL z. P z (pi_1 o ... o pi_n o t))             *)
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
    96
(* or    id (ALL z. P z (pi_1 o ... o pi_n o t))                     *)
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
    97
(*                                                                   *)
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
    98
(* where "id" protects the subformula from simplification            *)
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
    99
(*********************************************************************)
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   100
69597
ff784d5a5bfb isabelle update -u control_cartouches;
wenzelm
parents: 67522
diff changeset
   101
fun inst_conj_all names ps pis (Const (\<^const_name>\<open>HOL.conj\<close>, _) $ p $ q) _ =
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   102
      (case head_of p of
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   103
         Const (name, _) =>
36692
54b64d4ad524 farewell to old-style mem infixes -- type inference in situations with mem_int and mem_string should provide enough information to resolve the type of (op =)
haftmann
parents: 36428
diff changeset
   104
           if member (op =) names name then SOME (HOLogic.mk_conj (p,
69597
ff784d5a5bfb isabelle update -u control_cartouches;
wenzelm
parents: 67522
diff changeset
   105
             Const (\<^const_name>\<open>Fun.id\<close>, HOLogic.boolT --> HOLogic.boolT) $
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   106
               (subst_bounds (pis, strip_all pis q))))
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   107
           else NONE
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   108
       | _ => NONE)
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   109
  | inst_conj_all names ps pis t u =
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   110
      if member (op aconv) ps (head_of u) then
69597
ff784d5a5bfb isabelle update -u control_cartouches;
wenzelm
parents: 67522
diff changeset
   111
        SOME (Const (\<^const_name>\<open>Fun.id\<close>, HOLogic.boolT --> HOLogic.boolT) $
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   112
          (subst_bounds (pis, strip_all pis t)))
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   113
      else NONE
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   114
  | inst_conj_all _ _ _ _ _ = NONE;
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   115
51717
9e7d1c139569 simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents: 50771
diff changeset
   116
fun inst_conj_all_tac ctxt k = EVERY
60754
02924903a6fd prefer tactics with explicit context;
wenzelm
parents: 60642
diff changeset
   117
  [TRY (EVERY [eresolve_tac ctxt [conjE] 1, resolve_tac ctxt [conjI] 1, assume_tac ctxt 1]),
02924903a6fd prefer tactics with explicit context;
wenzelm
parents: 60642
diff changeset
   118
   REPEAT_DETERM_N k (eresolve_tac ctxt [allE] 1),
51717
9e7d1c139569 simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents: 50771
diff changeset
   119
   simp_tac (put_simpset HOL_basic_ss ctxt addsimps [@{thm id_apply}]) 1];
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   120
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   121
fun map_term f t u = (case f t u of
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   122
      NONE => map_term' f t u | x => x)
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   123
and map_term' f (t $ u) (t' $ u') = (case (map_term f t t', map_term f u u') of
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   124
      (NONE, NONE) => NONE
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   125
    | (SOME t'', NONE) => SOME (t'' $ u)
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   126
    | (NONE, SOME u'') => SOME (t $ u'')
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   127
    | (SOME t'', SOME u'') => SOME (t'' $ u''))
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   128
  | map_term' f (Abs (s, T, t)) (Abs (s', T', t')) = (case map_term f t t' of
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   129
      NONE => NONE
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   130
    | SOME t'' => SOME (Abs (s, T, t'')))
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   131
  | map_term' _ _ _ = NONE;
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   132
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   133
(*********************************************************************)
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   134
(*         Prove  F[f t]  from  F[t],  where F is monotone           *)
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   135
(*********************************************************************)
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   136
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   137
fun map_thm ctxt f tac monos opt th =
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   138
  let
59582
0fbed69ff081 tuned signature -- prefer qualified names;
wenzelm
parents: 59498
diff changeset
   139
    val prop = Thm.prop_of th;
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   140
    fun prove t =
74524
8ee3d5d3c1bf more accurate treatment of context, notably for nested Goal.proof / SUBPROOF;
wenzelm
parents: 74523
diff changeset
   141
      Goal.prove ctxt [] [] t (fn {context = goal_ctxt, ...} =>
8ee3d5d3c1bf more accurate treatment of context, notably for nested Goal.proof / SUBPROOF;
wenzelm
parents: 74523
diff changeset
   142
        EVERY [cut_facts_tac [th] 1, eresolve_tac goal_ctxt [rev_mp] 1,
8ee3d5d3c1bf more accurate treatment of context, notably for nested Goal.proof / SUBPROOF;
wenzelm
parents: 74523
diff changeset
   143
          REPEAT_DETERM (FIRSTGOAL (resolve_tac goal_ctxt monos)),
8ee3d5d3c1bf more accurate treatment of context, notably for nested Goal.proof / SUBPROOF;
wenzelm
parents: 74523
diff changeset
   144
          REPEAT_DETERM (resolve_tac goal_ctxt [impI] 1 THEN (assume_tac goal_ctxt 1 ORELSE tac))])
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   145
  in Option.map prove (map_term f prop (the_default prop opt)) end;
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   146
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   147
fun abs_params params t =
29276
94b1ffec9201 qualified Term.rename_wrt_term;
wenzelm
parents: 29270
diff changeset
   148
  let val vs =  map (Var o apfst (rpair 0)) (Term.rename_wrt_term t params)
46218
ecf6375e2abb renamed Term.list_all to Logic.list_all, in accordance to HOLogic.list_all;
wenzelm
parents: 44929
diff changeset
   149
  in (Logic.list_all (params, t), (rev vs, subst_bounds (vs, t))) end;
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   150
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   151
fun inst_params thy (vs, p) th cts =
59582
0fbed69ff081 tuned signature -- prefer qualified names;
wenzelm
parents: 59498
diff changeset
   152
  let val env = Pattern.first_order_match thy (p, Thm.prop_of th)
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   153
    (Vartab.empty, Vartab.empty)
74282
c2ee8d993d6a clarified signature: more scalable operations;
wenzelm
parents: 70326
diff changeset
   154
  in
c2ee8d993d6a clarified signature: more scalable operations;
wenzelm
parents: 70326
diff changeset
   155
    Thm.instantiate (TVars.empty, Vars.make (map (dest_Var o Envir.subst_term env) vs ~~ cts)) th
c2ee8d993d6a clarified signature: more scalable operations;
wenzelm
parents: 70326
diff changeset
   156
  end;
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   157
74523
wenzelm
parents: 74522
diff changeset
   158
fun prove_strong_ind s alt_name avoids lthy =
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   159
  let
74523
wenzelm
parents: 74522
diff changeset
   160
    val thy = Proof_Context.theory_of lthy;
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   161
    val ({names, ...}, {raw_induct, intrs, elims, ...}) =
74523
wenzelm
parents: 74522
diff changeset
   162
      Inductive.the_inductive_global lthy (Sign.intern_const thy s);
31723
f5cafe803b55 discontinued ancient tradition to suffix certain ML module names with "_package"
haftmann
parents: 31177
diff changeset
   163
    val ind_params = Inductive.params_of raw_induct;
74523
wenzelm
parents: 74522
diff changeset
   164
    val raw_induct = atomize_induct lthy raw_induct;
wenzelm
parents: 74522
diff changeset
   165
    val elims = map (atomize_induct lthy) elims;
wenzelm
parents: 74522
diff changeset
   166
    val monos = Inductive.get_monos lthy;
wenzelm
parents: 74522
diff changeset
   167
    val eqvt_thms = NominalThmDecls.get_eqvt_thms lthy;
33040
cffdb7b28498 removed old-style \ and \\ infixes
haftmann
parents: 33038
diff changeset
   168
    val _ = (case subtract (op =) (fold (Term.add_const_names o Thm.prop_of) eqvt_thms []) names of
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   169
        [] => ()
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   170
      | xs => error ("Missing equivariance theorem for predicate(s): " ^
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   171
          commas_quote xs));
44045
2814ff2a6e3e infrastructure for attaching names to hypothesis in cases; realised via the same tag mechanism as case names
nipkow
parents: 43326
diff changeset
   172
    val induct_cases = map (fst o fst) (fst (Rule_Cases.get (the
74523
wenzelm
parents: 74522
diff changeset
   173
      (Induct.lookup_inductP lthy (hd names)))));
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   174
    val induct_cases' = if null induct_cases then replicate (length intrs) ""
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   175
      else induct_cases;
74523
wenzelm
parents: 74522
diff changeset
   176
    val (raw_induct', ctxt') = lthy
70326
wenzelm
parents: 69597
diff changeset
   177
      |> yield_singleton (Variable.import_terms false) (Thm.prop_of raw_induct);
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   178
    val concls = raw_induct' |> Logic.strip_imp_concl |> HOLogic.dest_Trueprop |>
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   179
      HOLogic.dest_conj |> map (HOLogic.dest_imp ##> strip_comb);
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   180
    val ps = map (fst o snd) concls;
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   181
59058
a78612c67ec0 renamed "pairself" to "apply2", in accordance to @{apply 2};
wenzelm
parents: 58112
diff changeset
   182
    val _ = (case duplicates (op = o apply2 fst) avoids of
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   183
        [] => ()
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   184
      | xs => error ("Duplicate case names: " ^ commas_quote (map fst xs)));
33040
cffdb7b28498 removed old-style \ and \\ infixes
haftmann
parents: 33038
diff changeset
   185
    val _ = (case subtract (op =) induct_cases (map fst avoids) of
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   186
        [] => ()
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   187
      | xs => error ("No such case(s) in inductive definition: " ^ commas_quote xs));
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   188
    fun mk_avoids params name sets =
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   189
      let
42361
23f352990944 modernized structure Proof_Context;
wenzelm
parents: 41228
diff changeset
   190
        val (_, ctxt') = Proof_Context.add_fixes
74523
wenzelm
parents: 74522
diff changeset
   191
          (map (fn (s, T) => (Binding.name s, SOME T, NoSyn)) params) lthy;
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   192
        fun mk s =
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   193
          let
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   194
            val t = Syntax.read_term ctxt' s;
44241
7943b69f0188 modernized signature of Term.absfree/absdummy;
wenzelm
parents: 44045
diff changeset
   195
            val t' = fold_rev absfree params t |>
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   196
              funpow (length params) (fn Abs (_, _, t) => t)
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   197
          in (t', HOLogic.dest_setT (fastype_of t)) end
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   198
          handle TERM _ =>
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   199
            error ("Expression " ^ quote s ^ " to be avoided in case " ^
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   200
              quote name ^ " is not a set type");
30108
bd78f08b0ba1 Added postprocessing rules for fresh_star.
berghofe
parents: 30087
diff changeset
   201
        fun add_set p [] = [p]
bd78f08b0ba1 Added postprocessing rules for fresh_star.
berghofe
parents: 30087
diff changeset
   202
          | add_set (t, T) ((u, U) :: ps) =
bd78f08b0ba1 Added postprocessing rules for fresh_star.
berghofe
parents: 30087
diff changeset
   203
              if T = U then
bd78f08b0ba1 Added postprocessing rules for fresh_star.
berghofe
parents: 30087
diff changeset
   204
                let val S = HOLogic.mk_setT T
69597
ff784d5a5bfb isabelle update -u control_cartouches;
wenzelm
parents: 67522
diff changeset
   205
                in (Const (\<^const_name>\<open>sup\<close>, S --> S --> S) $ u $ t, T) :: ps
30108
bd78f08b0ba1 Added postprocessing rules for fresh_star.
berghofe
parents: 30087
diff changeset
   206
                end
bd78f08b0ba1 Added postprocessing rules for fresh_star.
berghofe
parents: 30087
diff changeset
   207
              else (u, U) :: add_set (t, T) ps
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   208
      in
30108
bd78f08b0ba1 Added postprocessing rules for fresh_star.
berghofe
parents: 30087
diff changeset
   209
        fold (mk #> add_set) sets []
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   210
      end;
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   211
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   212
    val prems = map (fn (prem, name) =>
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   213
      let
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   214
        val prems = map (incr_boundvars 1) (Logic.strip_assums_hyp prem);
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   215
        val concl = incr_boundvars 1 (Logic.strip_assums_concl prem);
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   216
        val params = Logic.strip_params prem
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   217
      in
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   218
        (params,
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   219
         if null avoids then
30450
7655e6533209 HOLogic.mk_set, HOLogic.dest_set
haftmann
parents: 30364
diff changeset
   220
           map (fn (T, ts) => (HOLogic.mk_set T ts, T))
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   221
             (fold (add_binders thy 0) (prems @ [concl]) [])
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   222
         else case AList.lookup op = avoids name of
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   223
           NONE => []
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   224
         | SOME sets =>
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   225
             map (apfst (incr_boundvars 1)) (mk_avoids params name sets),
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   226
         prems, strip_comb (HOLogic.dest_Trueprop concl))
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   227
      end) (Logic.strip_imp_prems raw_induct' ~~ induct_cases');
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   228
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   229
    val atomTs = distinct op = (maps (map snd o #2) prems);
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   230
    val atoms = map (fst o dest_Type) atomTs;
69597
ff784d5a5bfb isabelle update -u control_cartouches;
wenzelm
parents: 67522
diff changeset
   231
    val ind_sort = if null atomTs then \<^sort>\<open>type\<close>
36428
874843c1e96e really minimize sorts after certification -- looks like this is intended here;
wenzelm
parents: 36323
diff changeset
   232
      else Sign.minimize_sort thy (Sign.certify_sort thy (map (fn a => Sign.intern_class thy
874843c1e96e really minimize sorts after certification -- looks like this is intended here;
wenzelm
parents: 36323
diff changeset
   233
        ("fs_" ^ Long_Name.base_name a)) atoms));
43326
47cf4bc789aa simplified Name.variant -- discontinued builtin fold_map;
wenzelm
parents: 42361
diff changeset
   234
    val (fs_ctxt_tyname, _) = Name.variant "'n" (Variable.names_of ctxt');
30087
a780642a9c9c nominal_inductive and equivariance now work on local_theory.
berghofe
parents: 29585
diff changeset
   235
    val ([fs_ctxt_name], ctxt'') = Variable.variant_fixes ["z"] ctxt';
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   236
    val fsT = TFree (fs_ctxt_tyname, ind_sort);
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   237
60801
7664e0916eec tuned signature;
wenzelm
parents: 60787
diff changeset
   238
    val inductive_forall_def' = Thm.instantiate'
59621
291934bac95e Thm.cterm_of and Thm.ctyp_of operate on local context;
wenzelm
parents: 59582
diff changeset
   239
      [SOME (Thm.global_ctyp_of thy fsT)] [] inductive_forall_def;
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   240
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   241
    fun lift_pred' t (Free (s, T)) ts =
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   242
      list_comb (Free (s, fsT --> T), t :: ts);
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   243
    val lift_pred = lift_pred' (Bound 0);
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   244
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   245
    fun lift_prem (t as (f $ u)) =
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   246
          let val (p, ts) = strip_comb t
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   247
          in
44868
92be5b32ca71 more modularization
haftmann
parents: 44689
diff changeset
   248
            if member (op =) ps p then HOLogic.mk_induct_forall fsT $
92be5b32ca71 more modularization
haftmann
parents: 44689
diff changeset
   249
              Abs ("z", fsT, lift_pred p (map (incr_boundvars 1) ts))
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   250
            else lift_prem f $ lift_prem u
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   251
          end
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   252
      | lift_prem (Abs (s, T, t)) = Abs (s, T, lift_prem t)
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   253
      | lift_prem t = t;
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   254
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   255
    fun mk_fresh (x, T) = HOLogic.mk_Trueprop
31938
f193d95b4632 nominal.ML is nominal_datatype.ML
haftmann
parents: 31723
diff changeset
   256
      (NominalDatatype.fresh_star_const T fsT $ x $ Bound 0);
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   257
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   258
    val (prems', prems'') = split_list (map (fn (params, sets, prems, (p, ts)) =>
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   259
      let
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   260
        val params' = params @ [("y", fsT)];
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   261
        val prem = Logic.list_implies
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   262
          (map mk_fresh sets @
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   263
           map (fn prem =>
30087
a780642a9c9c nominal_inductive and equivariance now work on local_theory.
berghofe
parents: 29585
diff changeset
   264
             if null (preds_of ps prem) then prem
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   265
             else lift_prem prem) prems,
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   266
           HOLogic.mk_Trueprop (lift_pred p ts));
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   267
      in abs_params params' prem end) prems);
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   268
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   269
    val ind_vars =
58112
8081087096ad renamed modules defining old datatypes, as a step towards having 'datatype_new' take 'datatype's place
blanchet
parents: 56253
diff changeset
   270
      (Old_Datatype_Prop.indexify_names (replicate (length atomTs) "pi") ~~
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   271
       map NominalAtoms.mk_permT atomTs) @ [("z", fsT)];
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   272
    val ind_Ts = rev (map snd ind_vars);
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   273
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   274
    val concl = HOLogic.mk_Trueprop (foldr1 HOLogic.mk_conj
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   275
      (map (fn (prem, (p, ts)) => HOLogic.mk_imp (prem,
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   276
        HOLogic.list_all (ind_vars, lift_pred p
31938
f193d95b4632 nominal.ML is nominal_datatype.ML
haftmann
parents: 31723
diff changeset
   277
          (map (fold_rev (NominalDatatype.mk_perm ind_Ts)
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   278
            (map Bound (length atomTs downto 1))) ts)))) concls));
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   279
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   280
    val concl' = HOLogic.mk_Trueprop (foldr1 HOLogic.mk_conj
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   281
      (map (fn (prem, (p, ts)) => HOLogic.mk_imp (prem,
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   282
        lift_pred' (Free (fs_ctxt_name, fsT)) p ts)) concls));
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   283
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   284
    val (vc_compat, vc_compat') = map (fn (params, sets, prems, (p, ts)) =>
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   285
      map (fn q => abs_params params (incr_boundvars ~1 (Logic.list_implies
32952
aeb1e44fbc19 replaced String.concat by implode;
wenzelm
parents: 32304
diff changeset
   286
          (map_filter (fn prem =>
30087
a780642a9c9c nominal_inductive and equivariance now work on local_theory.
berghofe
parents: 29585
diff changeset
   287
             if null (preds_of ps prem) then SOME prem
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   288
             else map_term (split_conj (K o I) names) prem prem) prems, q))))
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   289
        (maps (fn (t, T) => map (fn (u, U) => HOLogic.mk_Trueprop
31938
f193d95b4632 nominal.ML is nominal_datatype.ML
haftmann
parents: 31723
diff changeset
   290
           (NominalDatatype.fresh_star_const U T $ u $ t)) sets)
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   291
             (ts ~~ binder_types (fastype_of p)) @
69597
ff784d5a5bfb isabelle update -u control_cartouches;
wenzelm
parents: 67522
diff changeset
   292
         map (fn (u, U) => HOLogic.mk_Trueprop (Const (\<^const_name>\<open>finite\<close>,
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   293
           HOLogic.mk_setT U --> HOLogic.boolT) $ u)) sets) |>
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   294
      split_list) prems |> split_list;
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   295
39557
fe5722fce758 renamed structure PureThy to Pure_Thy and moved most content to Global_Theory, to emphasize that this is global-only;
wenzelm
parents: 39159
diff changeset
   296
    val perm_pi_simp = Global_Theory.get_thms thy "perm_pi_simp";
fe5722fce758 renamed structure PureThy to Pure_Thy and moved most content to Global_Theory, to emphasize that this is global-only;
wenzelm
parents: 39159
diff changeset
   297
    val pt2_atoms = map (fn a => Global_Theory.get_thm thy
30364
577edc39b501 moved basic algebra of long names from structure NameSpace to Long_Name;
wenzelm
parents: 30307
diff changeset
   298
      ("pt_" ^ Long_Name.base_name a ^ "2")) atoms;
74524
8ee3d5d3c1bf more accurate treatment of context, notably for nested Goal.proof / SUBPROOF;
wenzelm
parents: 74523
diff changeset
   299
    fun eqvt_ss ctxt =
8ee3d5d3c1bf more accurate treatment of context, notably for nested Goal.proof / SUBPROOF;
wenzelm
parents: 74523
diff changeset
   300
      put_simpset HOL_basic_ss ctxt
8ee3d5d3c1bf more accurate treatment of context, notably for nested Goal.proof / SUBPROOF;
wenzelm
parents: 74523
diff changeset
   301
        addsimps (eqvt_thms @ perm_pi_simp @ pt2_atoms)
8ee3d5d3c1bf more accurate treatment of context, notably for nested Goal.proof / SUBPROOF;
wenzelm
parents: 74523
diff changeset
   302
        addsimprocs [mk_perm_bool_simproc [\<^const_name>\<open>Fun.id\<close>],
78806
aca84704d46f more standard simproc_setup using ML antiquotation;
wenzelm
parents: 78095
diff changeset
   303
          NominalPermeq.perm_app_simproc, NominalPermeq.perm_fun_simproc];
39557
fe5722fce758 renamed structure PureThy to Pure_Thy and moved most content to Global_Theory, to emphasize that this is global-only;
wenzelm
parents: 39159
diff changeset
   304
    val fresh_star_bij = Global_Theory.get_thms thy "fresh_star_bij";
28730
71c946ce7eb9 Streamlined functions for accessing information about atoms.
berghofe
parents: 28653
diff changeset
   305
    val pt_insts = map (NominalAtoms.pt_inst_of thy) atoms;
71c946ce7eb9 Streamlined functions for accessing information about atoms.
berghofe
parents: 28653
diff changeset
   306
    val at_insts = map (NominalAtoms.at_inst_of thy) atoms;
71c946ce7eb9 Streamlined functions for accessing information about atoms.
berghofe
parents: 28653
diff changeset
   307
    val dj_thms = maps (fn a =>
33040
cffdb7b28498 removed old-style \ and \\ infixes
haftmann
parents: 33038
diff changeset
   308
      map (NominalAtoms.dj_thm_of thy a) (remove (op =) a atoms)) atoms;
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   309
    val finite_ineq = map2 (fn th => fn th' => th' RS (th RS
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   310
      @{thm pt_set_finite_ineq})) pt_insts at_insts;
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   311
    val perm_set_forget =
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   312
      map (fn th => th RS @{thm dj_perm_set_forget}) dj_thms;
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   313
    val perm_freshs_freshs = atomTs ~~ map2 (fn th => fn th' => th' RS (th RS
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   314
      @{thm pt_freshs_freshs})) pt_insts at_insts;
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   315
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   316
    fun obtain_fresh_name ts sets (T, fin) (freshs, ths1, ths2, ths3, ctxt) =
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   317
      let
42361
23f352990944 modernized structure Proof_Context;
wenzelm
parents: 41228
diff changeset
   318
        val thy = Proof_Context.theory_of ctxt;
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   319
        (** protect terms to avoid that fresh_star_prod_set interferes with  **)
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   320
        (** pairs used in introduction rules of inductive predicate          **)
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   321
        fun protect t =
69597
ff784d5a5bfb isabelle update -u control_cartouches;
wenzelm
parents: 67522
diff changeset
   322
          let val T = fastype_of t in Const (\<^const_name>\<open>Fun.id\<close>, T --> T) $ t end;
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   323
        val p = foldr1 HOLogic.mk_prod (map protect ts);
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   324
        val atom = fst (dest_Type T);
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   325
        val {at_inst, ...} = NominalAtoms.the_atom_info thy atom;
39557
fe5722fce758 renamed structure PureThy to Pure_Thy and moved most content to Global_Theory, to emphasize that this is global-only;
wenzelm
parents: 39159
diff changeset
   326
        val fs_atom = Global_Theory.get_thm thy
30364
577edc39b501 moved basic algebra of long names from structure NameSpace to Long_Name;
wenzelm
parents: 30307
diff changeset
   327
          ("fs_" ^ Long_Name.base_name atom ^ "1");
60801
7664e0916eec tuned signature;
wenzelm
parents: 60787
diff changeset
   328
        val avoid_th = Thm.instantiate'
59621
291934bac95e Thm.cterm_of and Thm.ctyp_of operate on local context;
wenzelm
parents: 59582
diff changeset
   329
          [SOME (Thm.global_ctyp_of thy (fastype_of p))] [SOME (Thm.global_cterm_of thy p)]
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   330
          ([at_inst, fin, fs_atom] MRS @{thm at_set_avoiding});
32202
443d5cfaba1b SUBPROOF/Obtain.result: named params;
wenzelm
parents: 32172
diff changeset
   331
        val (([(_, cx)], th1 :: th2 :: ths), ctxt') = Obtain.result
51717
9e7d1c139569 simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents: 50771
diff changeset
   332
          (fn ctxt' => EVERY
60754
02924903a6fd prefer tactics with explicit context;
wenzelm
parents: 60642
diff changeset
   333
            [resolve_tac ctxt' [avoid_th] 1,
51717
9e7d1c139569 simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents: 50771
diff changeset
   334
             full_simp_tac (put_simpset HOL_ss ctxt' addsimps [@{thm fresh_star_prod_set}]) 1,
9e7d1c139569 simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents: 50771
diff changeset
   335
             full_simp_tac (put_simpset HOL_basic_ss ctxt' addsimps [@{thm id_apply}]) 1,
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   336
             rotate_tac 1 1,
60754
02924903a6fd prefer tactics with explicit context;
wenzelm
parents: 60642
diff changeset
   337
             REPEAT (eresolve_tac ctxt' [conjE] 1)])
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   338
          [] ctxt;
67522
9e712280cc37 clarified take/drop/chop prefix/suffix;
wenzelm
parents: 67405
diff changeset
   339
        val (Ts1, _ :: Ts2) = chop_prefix (not o equal T) (map snd sets);
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   340
        val pTs = map NominalAtoms.mk_permT (Ts1 @ Ts2);
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   341
        val (pis1, pis2) = chop (length Ts1)
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   342
          (map Bound (length pTs - 1 downto 0));
59582
0fbed69ff081 tuned signature -- prefer qualified names;
wenzelm
parents: 59498
diff changeset
   343
        val _ $ (f $ (_ $ pi $ l) $ r) = Thm.prop_of th2
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   344
        val th2' =
54983
2c57fc1f7a8c more accurate context;
wenzelm
parents: 54895
diff changeset
   345
          Goal.prove ctxt' [] []
46218
ecf6375e2abb renamed Term.list_all to Logic.list_all, in accordance to HOLogic.list_all;
wenzelm
parents: 44929
diff changeset
   346
            (Logic.list_all (map (pair "pi") pTs, HOLogic.mk_Trueprop
31938
f193d95b4632 nominal.ML is nominal_datatype.ML
haftmann
parents: 31723
diff changeset
   347
               (f $ fold_rev (NominalDatatype.mk_perm (rev pTs))
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   348
                  (pis1 @ pi :: pis2) l $ r)))
74524
8ee3d5d3c1bf more accurate treatment of context, notably for nested Goal.proof / SUBPROOF;
wenzelm
parents: 74523
diff changeset
   349
            (fn {context = goal_ctxt, ...} =>
8ee3d5d3c1bf more accurate treatment of context, notably for nested Goal.proof / SUBPROOF;
wenzelm
parents: 74523
diff changeset
   350
              cut_facts_tac [th2] 1 THEN
8ee3d5d3c1bf more accurate treatment of context, notably for nested Goal.proof / SUBPROOF;
wenzelm
parents: 74523
diff changeset
   351
              full_simp_tac (put_simpset HOL_basic_ss goal_ctxt addsimps perm_set_forget) 1) |>
8ee3d5d3c1bf more accurate treatment of context, notably for nested Goal.proof / SUBPROOF;
wenzelm
parents: 74523
diff changeset
   352
          Simplifier.simplify (eqvt_ss ctxt')
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   353
      in
59582
0fbed69ff081 tuned signature -- prefer qualified names;
wenzelm
parents: 59498
diff changeset
   354
        (freshs @ [Thm.term_of cx],
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   355
         ths1 @ ths, ths2 @ [th1], ths3 @ [th2'], ctxt')
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   356
      end;
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   357
74524
8ee3d5d3c1bf more accurate treatment of context, notably for nested Goal.proof / SUBPROOF;
wenzelm
parents: 74523
diff changeset
   358
    fun mk_ind_proof ctxt thss =
8ee3d5d3c1bf more accurate treatment of context, notably for nested Goal.proof / SUBPROOF;
wenzelm
parents: 74523
diff changeset
   359
      Goal.prove ctxt [] prems' concl' (fn {prems = ihyps, context = goal_ctxt} =>
8ee3d5d3c1bf more accurate treatment of context, notably for nested Goal.proof / SUBPROOF;
wenzelm
parents: 74523
diff changeset
   360
        let val th = Goal.prove goal_ctxt [] [] concl (fn {context = goal_ctxt1, ...} =>
8ee3d5d3c1bf more accurate treatment of context, notably for nested Goal.proof / SUBPROOF;
wenzelm
parents: 74523
diff changeset
   361
          resolve_tac goal_ctxt1 [raw_induct] 1 THEN
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   362
          EVERY (maps (fn (((((_, sets, oprems, _),
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   363
              vc_compat_ths), vc_compat_vs), ihyp), vs_ihypt) =>
74524
8ee3d5d3c1bf more accurate treatment of context, notably for nested Goal.proof / SUBPROOF;
wenzelm
parents: 74523
diff changeset
   364
            [REPEAT (resolve_tac goal_ctxt1 [allI] 1), simp_tac (eqvt_ss goal_ctxt1) 1,
8ee3d5d3c1bf more accurate treatment of context, notably for nested Goal.proof / SUBPROOF;
wenzelm
parents: 74523
diff changeset
   365
             SUBPROOF (fn {prems = gprems, params, concl, context = goal_ctxt2, ...} =>
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   366
               let
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   367
                 val (cparams', (pis, z)) =
32202
443d5cfaba1b SUBPROOF/Obtain.result: named params;
wenzelm
parents: 32172
diff changeset
   368
                   chop (length params - length atomTs - 1) (map #2 params) ||>
59582
0fbed69ff081 tuned signature -- prefer qualified names;
wenzelm
parents: 59498
diff changeset
   369
                   (map Thm.term_of #> split_last);
0fbed69ff081 tuned signature -- prefer qualified names;
wenzelm
parents: 59498
diff changeset
   370
                 val params' = map Thm.term_of cparams'
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   371
                 val sets' = map (apfst (curry subst_bounds (rev params'))) sets;
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   372
                 val pi_sets = map (fn (t, _) =>
31938
f193d95b4632 nominal.ML is nominal_datatype.ML
haftmann
parents: 31723
diff changeset
   373
                   fold_rev (NominalDatatype.mk_perm []) pis t) sets';
59582
0fbed69ff081 tuned signature -- prefer qualified names;
wenzelm
parents: 59498
diff changeset
   374
                 val (P, ts) = strip_comb (HOLogic.dest_Trueprop (Thm.term_of concl));
32952
aeb1e44fbc19 replaced String.concat by implode;
wenzelm
parents: 32304
diff changeset
   375
                 val gprems1 = map_filter (fn (th, t) =>
30087
a780642a9c9c nominal_inductive and equivariance now work on local_theory.
berghofe
parents: 29585
diff changeset
   376
                   if null (preds_of ps t) then SOME th
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   377
                   else
74524
8ee3d5d3c1bf more accurate treatment of context, notably for nested Goal.proof / SUBPROOF;
wenzelm
parents: 74523
diff changeset
   378
                     map_thm goal_ctxt2 (split_conj (K o I) names)
8ee3d5d3c1bf more accurate treatment of context, notably for nested Goal.proof / SUBPROOF;
wenzelm
parents: 74523
diff changeset
   379
                       (eresolve_tac goal_ctxt2 [conjunct1] 1) monos NONE th)
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   380
                   (gprems ~~ oprems);
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   381
                 val vc_compat_ths' = map2 (fn th => fn p =>
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   382
                   let
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   383
                     val th' = gprems1 MRS inst_params thy p th cparams';
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   384
                     val (h, ts) =
59582
0fbed69ff081 tuned signature -- prefer qualified names;
wenzelm
parents: 59498
diff changeset
   385
                       strip_comb (HOLogic.dest_Trueprop (Thm.concl_of th'))
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   386
                   in
74524
8ee3d5d3c1bf more accurate treatment of context, notably for nested Goal.proof / SUBPROOF;
wenzelm
parents: 74523
diff changeset
   387
                     Goal.prove goal_ctxt2 [] []
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   388
                       (HOLogic.mk_Trueprop (list_comb (h,
31938
f193d95b4632 nominal.ML is nominal_datatype.ML
haftmann
parents: 31723
diff changeset
   389
                          map (fold_rev (NominalDatatype.mk_perm []) pis) ts)))
74524
8ee3d5d3c1bf more accurate treatment of context, notably for nested Goal.proof / SUBPROOF;
wenzelm
parents: 74523
diff changeset
   390
                       (fn {context = goal_ctxt3, ...} =>
8ee3d5d3c1bf more accurate treatment of context, notably for nested Goal.proof / SUBPROOF;
wenzelm
parents: 74523
diff changeset
   391
                         simp_tac (put_simpset HOL_basic_ss goal_ctxt3 addsimps
8ee3d5d3c1bf more accurate treatment of context, notably for nested Goal.proof / SUBPROOF;
wenzelm
parents: 74523
diff changeset
   392
                          (fresh_star_bij @ finite_ineq)) 1 THEN resolve_tac goal_ctxt3 [th'] 1)
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   393
                   end) vc_compat_ths vc_compat_vs;
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   394
                 val (vc_compat_ths1, vc_compat_ths2) =
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   395
                   chop (length vc_compat_ths - length sets) vc_compat_ths';
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   396
                 val vc_compat_ths1' = map
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   397
                   (Conv.fconv_rule (Conv.arg_conv (Conv.arg_conv
74524
8ee3d5d3c1bf more accurate treatment of context, notably for nested Goal.proof / SUBPROOF;
wenzelm
parents: 74523
diff changeset
   398
                      (Simplifier.rewrite (eqvt_ss goal_ctxt2))))) vc_compat_ths1;
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   399
                 val (pis', fresh_ths1, fresh_ths2, fresh_ths3, ctxt'') = fold
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   400
                   (obtain_fresh_name ts sets)
74524
8ee3d5d3c1bf more accurate treatment of context, notably for nested Goal.proof / SUBPROOF;
wenzelm
parents: 74523
diff changeset
   401
                   (map snd sets' ~~ vc_compat_ths2) ([], [], [], [], goal_ctxt2);
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   402
                 fun concat_perm pi1 pi2 =
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   403
                   let val T = fastype_of pi1
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   404
                   in if T = fastype_of pi2 then
69597
ff784d5a5bfb isabelle update -u control_cartouches;
wenzelm
parents: 67522
diff changeset
   405
                       Const (\<^const_name>\<open>append\<close>, T --> T --> T) $ pi1 $ pi2
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   406
                     else pi2
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   407
                   end;
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   408
                 val pis'' = fold_rev (concat_perm #> map) pis' pis;
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   409
                 val ihyp' = inst_params thy vs_ihypt ihyp
31938
f193d95b4632 nominal.ML is nominal_datatype.ML
haftmann
parents: 31723
diff changeset
   410
                   (map (fold_rev (NominalDatatype.mk_perm [])
59621
291934bac95e Thm.cterm_of and Thm.ctyp_of operate on local context;
wenzelm
parents: 59582
diff changeset
   411
                      (pis' @ pis) #> Thm.global_cterm_of thy) params' @ [Thm.global_cterm_of thy z]);
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   412
                 fun mk_pi th =
74524
8ee3d5d3c1bf more accurate treatment of context, notably for nested Goal.proof / SUBPROOF;
wenzelm
parents: 74523
diff changeset
   413
                   Simplifier.simplify
8ee3d5d3c1bf more accurate treatment of context, notably for nested Goal.proof / SUBPROOF;
wenzelm
parents: 74523
diff changeset
   414
                     (put_simpset HOL_basic_ss ctxt'' addsimps [@{thm id_apply}]
31938
f193d95b4632 nominal.ML is nominal_datatype.ML
haftmann
parents: 31723
diff changeset
   415
                       addsimprocs [NominalDatatype.perm_simproc])
74524
8ee3d5d3c1bf more accurate treatment of context, notably for nested Goal.proof / SUBPROOF;
wenzelm
parents: 74523
diff changeset
   416
                     (Simplifier.simplify (eqvt_ss ctxt'')
8ee3d5d3c1bf more accurate treatment of context, notably for nested Goal.proof / SUBPROOF;
wenzelm
parents: 74523
diff changeset
   417
                       (fold_rev (mk_perm_bool ctxt'' o Thm.cterm_of ctxt'')
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   418
                         (pis' @ pis) th));
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   419
                 val gprems2 = map (fn (th, t) =>
30087
a780642a9c9c nominal_inductive and equivariance now work on local_theory.
berghofe
parents: 29585
diff changeset
   420
                   if null (preds_of ps t) then mk_pi th
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   421
                   else
74524
8ee3d5d3c1bf more accurate treatment of context, notably for nested Goal.proof / SUBPROOF;
wenzelm
parents: 74523
diff changeset
   422
                     mk_pi (the (map_thm ctxt'' (inst_conj_all names ps (rev pis''))
8ee3d5d3c1bf more accurate treatment of context, notably for nested Goal.proof / SUBPROOF;
wenzelm
parents: 74523
diff changeset
   423
                       (inst_conj_all_tac ctxt'' (length pis'')) monos (SOME t) th)))
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   424
                   (gprems ~~ oprems);
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   425
                 val perm_freshs_freshs' = map (fn (th, (_, T)) =>
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   426
                   th RS the (AList.lookup op = perm_freshs_freshs T))
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   427
                     (fresh_ths2 ~~ sets);
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   428
                 val th = Goal.prove ctxt'' [] []
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   429
                   (HOLogic.mk_Trueprop (list_comb (P $ hd ts,
31938
f193d95b4632 nominal.ML is nominal_datatype.ML
haftmann
parents: 31723
diff changeset
   430
                     map (fold_rev (NominalDatatype.mk_perm []) pis') (tl ts))))
74524
8ee3d5d3c1bf more accurate treatment of context, notably for nested Goal.proof / SUBPROOF;
wenzelm
parents: 74523
diff changeset
   431
                   (fn {context = goal_ctxt4, ...} =>
8ee3d5d3c1bf more accurate treatment of context, notably for nested Goal.proof / SUBPROOF;
wenzelm
parents: 74523
diff changeset
   432
                     EVERY ([simp_tac (eqvt_ss goal_ctxt4) 1,
8ee3d5d3c1bf more accurate treatment of context, notably for nested Goal.proof / SUBPROOF;
wenzelm
parents: 74523
diff changeset
   433
                     resolve_tac goal_ctxt4 [ihyp'] 1] @
8ee3d5d3c1bf more accurate treatment of context, notably for nested Goal.proof / SUBPROOF;
wenzelm
parents: 74523
diff changeset
   434
                     map (fn th => resolve_tac goal_ctxt4 [th] 1) fresh_ths3 @
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   435
                     [REPEAT_DETERM_N (length gprems)
74524
8ee3d5d3c1bf more accurate treatment of context, notably for nested Goal.proof / SUBPROOF;
wenzelm
parents: 74523
diff changeset
   436
                       (simp_tac (put_simpset HOL_basic_ss goal_ctxt4
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   437
                          addsimps [inductive_forall_def']
31938
f193d95b4632 nominal.ML is nominal_datatype.ML
haftmann
parents: 31723
diff changeset
   438
                          addsimprocs [NominalDatatype.perm_simproc]) 1 THEN
74524
8ee3d5d3c1bf more accurate treatment of context, notably for nested Goal.proof / SUBPROOF;
wenzelm
parents: 74523
diff changeset
   439
                        resolve_tac goal_ctxt4 gprems2 1)]));
59582
0fbed69ff081 tuned signature -- prefer qualified names;
wenzelm
parents: 59498
diff changeset
   440
                 val final = Goal.prove ctxt'' [] [] (Thm.term_of concl)
74524
8ee3d5d3c1bf more accurate treatment of context, notably for nested Goal.proof / SUBPROOF;
wenzelm
parents: 74523
diff changeset
   441
                   (fn {context = goal_ctxt5, ...} =>
8ee3d5d3c1bf more accurate treatment of context, notably for nested Goal.proof / SUBPROOF;
wenzelm
parents: 74523
diff changeset
   442
                     cut_facts_tac [th] 1 THEN full_simp_tac (put_simpset HOL_ss goal_ctxt5
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   443
                     addsimps vc_compat_ths1' @ fresh_ths1 @
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   444
                       perm_freshs_freshs') 1);
74524
8ee3d5d3c1bf more accurate treatment of context, notably for nested Goal.proof / SUBPROOF;
wenzelm
parents: 74523
diff changeset
   445
                 val final' = Proof_Context.export ctxt'' goal_ctxt2 [final];
8ee3d5d3c1bf more accurate treatment of context, notably for nested Goal.proof / SUBPROOF;
wenzelm
parents: 74523
diff changeset
   446
               in resolve_tac goal_ctxt2 final' 1 end) goal_ctxt1 1])
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   447
                 (prems ~~ thss ~~ vc_compat' ~~ ihyps ~~ prems'')))
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   448
        in
74524
8ee3d5d3c1bf more accurate treatment of context, notably for nested Goal.proof / SUBPROOF;
wenzelm
parents: 74523
diff changeset
   449
          cut_facts_tac [th] 1 THEN REPEAT (eresolve_tac goal_ctxt [conjE] 1) THEN
8ee3d5d3c1bf more accurate treatment of context, notably for nested Goal.proof / SUBPROOF;
wenzelm
parents: 74523
diff changeset
   450
          REPEAT (REPEAT (resolve_tac goal_ctxt [conjI, impI] 1) THEN
8ee3d5d3c1bf more accurate treatment of context, notably for nested Goal.proof / SUBPROOF;
wenzelm
parents: 74523
diff changeset
   451
            eresolve_tac goal_ctxt [impE] 1 THEN
8ee3d5d3c1bf more accurate treatment of context, notably for nested Goal.proof / SUBPROOF;
wenzelm
parents: 74523
diff changeset
   452
            assume_tac goal_ctxt 1 THEN REPEAT (eresolve_tac goal_ctxt @{thms allE_Nil} 1) THEN
8ee3d5d3c1bf more accurate treatment of context, notably for nested Goal.proof / SUBPROOF;
wenzelm
parents: 74523
diff changeset
   453
            asm_full_simp_tac goal_ctxt 1)
30108
bd78f08b0ba1 Added postprocessing rules for fresh_star.
berghofe
parents: 30087
diff changeset
   454
        end) |>
74524
8ee3d5d3c1bf more accurate treatment of context, notably for nested Goal.proof / SUBPROOF;
wenzelm
parents: 74523
diff changeset
   455
        fresh_postprocess ctxt |>
8ee3d5d3c1bf more accurate treatment of context, notably for nested Goal.proof / SUBPROOF;
wenzelm
parents: 74523
diff changeset
   456
        singleton (Proof_Context.export ctxt lthy);
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   457
  in
30087
a780642a9c9c nominal_inductive and equivariance now work on local_theory.
berghofe
parents: 29585
diff changeset
   458
    ctxt'' |>
74522
wenzelm
parents: 74282
diff changeset
   459
    Proof.theorem NONE (fn thss => fn lthy1 =>
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   460
      let
30364
577edc39b501 moved basic algebra of long names from structure NameSpace to Long_Name;
wenzelm
parents: 30307
diff changeset
   461
        val rec_name = space_implode "_" (map Long_Name.base_name names);
30223
24d975352879 renamed Binding.name_pos to Binding.make, renamed Binding.base_name to Binding.name_of, renamed Binding.map_base to Binding.map_name, added mandatory flag to Binding.qualify;
wenzelm
parents: 30108
diff changeset
   462
        val rec_qualified = Binding.qualify false rec_name;
33368
b1cf34f1855c modernized structure Rule_Cases;
wenzelm
parents: 33049
diff changeset
   463
        val ind_case_names = Rule_Cases.case_names induct_cases;
31723
f5cafe803b55 discontinued ancient tradition to suffix certain ML module names with "_package"
haftmann
parents: 31177
diff changeset
   464
        val induct_cases' = Inductive.partition_rules' raw_induct
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   465
          (intrs ~~ induct_cases); 
74522
wenzelm
parents: 74282
diff changeset
   466
        val thss' = map (map (atomize_intr lthy1)) thss;
31723
f5cafe803b55 discontinued ancient tradition to suffix certain ML module names with "_package"
haftmann
parents: 31177
diff changeset
   467
        val thsss = Inductive.partition_rules' raw_induct (intrs ~~ thss');
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   468
        val strong_raw_induct =
74522
wenzelm
parents: 74282
diff changeset
   469
          mk_ind_proof lthy1 thss' |> Inductive.rulify lthy1;
50771
2852f997bfb5 prefer negative "consumes", relative to the total number of prems, which is stable under more morphisms, notably those from nested context with assumes (cf. existing treatment of 'obtains');
wenzelm
parents: 46961
diff changeset
   470
        val strong_induct_atts =
78095
bc42c074e58f tuned signature: more position information;
wenzelm
parents: 74524
diff changeset
   471
          map (Attrib.internal \<^here> o K)
50771
2852f997bfb5 prefer negative "consumes", relative to the total number of prems, which is stable under more morphisms, notably those from nested context with assumes (cf. existing treatment of 'obtains');
wenzelm
parents: 46961
diff changeset
   472
            [ind_case_names, Rule_Cases.consumes (~ (Thm.nprems_of strong_raw_induct))];
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   473
        val strong_induct =
50771
2852f997bfb5 prefer negative "consumes", relative to the total number of prems, which is stable under more morphisms, notably those from nested context with assumes (cf. existing treatment of 'obtains');
wenzelm
parents: 46961
diff changeset
   474
          if length names > 1 then strong_raw_induct
2852f997bfb5 prefer negative "consumes", relative to the total number of prems, which is stable under more morphisms, notably those from nested context with assumes (cf. existing treatment of 'obtains');
wenzelm
parents: 46961
diff changeset
   475
          else strong_raw_induct RSN (2, rev_mp);
32304
berghofe
parents: 32303
diff changeset
   476
        val (induct_name, inducts_name) =
berghofe
parents: 32303
diff changeset
   477
          case alt_name of
32303
ba59e95a5d2b the derived induction principles can be given an explicit name
Christian Urban <urbanc@in.tum.de>
parents: 32202
diff changeset
   478
            NONE => (rec_qualified (Binding.name "strong_induct"),
ba59e95a5d2b the derived induction principles can be given an explicit name
Christian Urban <urbanc@in.tum.de>
parents: 32202
diff changeset
   479
                     rec_qualified (Binding.name "strong_inducts"))
32304
berghofe
parents: 32303
diff changeset
   480
          | SOME s => (Binding.name s, Binding.name (s ^ "s"));
74522
wenzelm
parents: 74282
diff changeset
   481
        val ((_, [strong_induct']), lthy2) = lthy1 |> Local_Theory.note
50771
2852f997bfb5 prefer negative "consumes", relative to the total number of prems, which is stable under more morphisms, notably those from nested context with assumes (cf. existing treatment of 'obtains');
wenzelm
parents: 46961
diff changeset
   482
          ((induct_name, strong_induct_atts), [strong_induct]);
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   483
        val strong_inducts =
74522
wenzelm
parents: 74282
diff changeset
   484
          Project_Rule.projects lthy2 (1 upto length names) strong_induct'
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   485
      in
74522
wenzelm
parents: 74282
diff changeset
   486
        lthy2 |>
50771
2852f997bfb5 prefer negative "consumes", relative to the total number of prems, which is stable under more morphisms, notably those from nested context with assumes (cf. existing treatment of 'obtains');
wenzelm
parents: 46961
diff changeset
   487
        Local_Theory.notes [((inducts_name, []),
2852f997bfb5 prefer negative "consumes", relative to the total number of prems, which is stable under more morphisms, notably those from nested context with assumes (cf. existing treatment of 'obtains');
wenzelm
parents: 46961
diff changeset
   488
          strong_inducts |> map (fn th => ([th],
78095
bc42c074e58f tuned signature: more position information;
wenzelm
parents: 74524
diff changeset
   489
            [Attrib.internal \<^here> (K ind_case_names),
bc42c074e58f tuned signature: more position information;
wenzelm
parents: 74524
diff changeset
   490
             Attrib.internal \<^here> (K (Rule_Cases.consumes (1 - Thm.nprems_of th)))])))] |> snd
30087
a780642a9c9c nominal_inductive and equivariance now work on local_theory.
berghofe
parents: 29585
diff changeset
   491
      end)
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   492
      (map (map (rulify_term thy #> rpair [])) vc_compat)
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   493
  end;
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   494
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   495
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   496
(* outer syntax *)
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   497
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   498
val _ =
69597
ff784d5a5bfb isabelle update -u control_cartouches;
wenzelm
parents: 67522
diff changeset
   499
  Outer_Syntax.local_theory_to_proof \<^command_keyword>\<open>nominal_inductive2\<close>
36960
01594f816e3a prefer structure Keyword, Parse, Parse_Spec, Outer_Syntax;
wenzelm
parents: 36692
diff changeset
   500
    "prove strong induction theorem for inductive predicate involving nominal datatypes"
62969
9f394a16c557 eliminated "xname" and variants;
wenzelm
parents: 62913
diff changeset
   501
    (Parse.name -- 
69597
ff784d5a5bfb isabelle update -u control_cartouches;
wenzelm
parents: 67522
diff changeset
   502
     Scan.option (\<^keyword>\<open>(\<close> |-- Parse.!!! (Parse.name --| \<^keyword>\<open>)\<close>)) --
ff784d5a5bfb isabelle update -u control_cartouches;
wenzelm
parents: 67522
diff changeset
   503
     (Scan.optional (\<^keyword>\<open>avoids\<close> |-- Parse.enum1 "|" (Parse.name --
ff784d5a5bfb isabelle update -u control_cartouches;
wenzelm
parents: 67522
diff changeset
   504
      (\<^keyword>\<open>:\<close> |-- Parse.and_list1 Parse.term))) []) >> (fn ((name, rule_name), avoids) =>
32303
ba59e95a5d2b the derived induction principles can be given an explicit name
Christian Urban <urbanc@in.tum.de>
parents: 32202
diff changeset
   505
        prove_strong_ind name rule_name avoids));
28653
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   506
4593c70e228e More general, still experimental version of nominal_inductive for
berghofe
parents:
diff changeset
   507
end