src/HOL/Tools/arith_data.ML
author paulson <lp15@cam.ac.uk>
Tue, 23 Apr 2024 10:26:04 +0100
changeset 80143 378593bf5109
parent 74561 8e6c973003c8
permissions -rw-r--r--
Tidying up another of the nominal examples
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
30878
309bfab064e9 tuned comment
haftmann
parents: 30722
diff changeset
     1
(*  Title:      HOL/Tools/arith_data.ML
24095
785c3cd7fcb5 moved lin_arith stuff to Tools/lin_arith.ML;
wenzelm
parents: 24076
diff changeset
     2
    Author:     Markus Wenzel, Stefan Berghofer, and Tobias Nipkow
9436
62bb04ab4b01 rearranged setup of arithmetic procedures, avoiding global reference values;
wenzelm
parents:
diff changeset
     3
33359
8b673ae1bf39 dedicated theory for loading numeral simprocs
haftmann
parents: 32957
diff changeset
     4
Common arithmetic proof auxiliary and legacy.
9436
62bb04ab4b01 rearranged setup of arithmetic procedures, avoiding global reference values;
wenzelm
parents:
diff changeset
     5
*)
62bb04ab4b01 rearranged setup of arithmetic procedures, avoiding global reference values;
wenzelm
parents:
diff changeset
     6
26101
a657683e902a tuned structures in arith_data.ML
haftmann
parents: 25484
diff changeset
     7
signature ARITH_DATA =
a657683e902a tuned structures in arith_data.ML
haftmann
parents: 25484
diff changeset
     8
sig
30686
47a32dd1b86e moved generic arith_tac (formerly silent_arith_tac), verbose_arith_tac (formerly arith_tac) to Arith_Data; simple_arith-tac now named linear_arith_tac
haftmann
parents: 30518
diff changeset
     9
  val arith_tac: Proof.context -> int -> tactic
59657
2441a80fb6c1 eliminated unused arith "verbose" flag -- tools that need options can use the context;
wenzelm
parents: 58820
diff changeset
    10
  val add_tactic: string -> (Proof.context -> int -> tactic) -> theory -> theory
30686
47a32dd1b86e moved generic arith_tac (formerly silent_arith_tac), verbose_arith_tac (formerly arith_tac) to Arith_Data; simple_arith-tac now named linear_arith_tac
haftmann
parents: 30518
diff changeset
    11
33359
8b673ae1bf39 dedicated theory for loading numeral simprocs
haftmann
parents: 32957
diff changeset
    12
  val mk_number: typ -> int -> term
8b673ae1bf39 dedicated theory for loading numeral simprocs
haftmann
parents: 32957
diff changeset
    13
  val mk_sum: typ -> term list -> term
8b673ae1bf39 dedicated theory for loading numeral simprocs
haftmann
parents: 32957
diff changeset
    14
  val long_mk_sum: typ -> term list -> term
8b673ae1bf39 dedicated theory for loading numeral simprocs
haftmann
parents: 32957
diff changeset
    15
  val dest_sum: term -> term list
8b673ae1bf39 dedicated theory for loading numeral simprocs
haftmann
parents: 32957
diff changeset
    16
30496
7cdcc9dd95cb vague cleanup in arith proof tools setup: deleted dead code, more proper structures, clearer arrangement
haftmann
parents: 29302
diff changeset
    17
  val prove_conv_nohyps: tactic list -> Proof.context -> term * term -> thm option
7cdcc9dd95cb vague cleanup in arith proof tools setup: deleted dead code, more proper structures, clearer arrangement
haftmann
parents: 29302
diff changeset
    18
  val prove_conv: tactic list -> Proof.context -> thm list -> term * term -> thm option
51717
9e7d1c139569 simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents: 50107
diff changeset
    19
  val prove_conv2: tactic -> (Proof.context -> tactic) -> Proof.context -> term * term -> thm
9e7d1c139569 simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents: 50107
diff changeset
    20
  val simp_all_tac: thm list -> Proof.context -> tactic
9e7d1c139569 simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents: 50107
diff changeset
    21
  val simplify_meta_eq: thm list -> Proof.context -> thm -> thm
26101
a657683e902a tuned structures in arith_data.ML
haftmann
parents: 25484
diff changeset
    22
end;
9436
62bb04ab4b01 rearranged setup of arithmetic procedures, avoiding global reference values;
wenzelm
parents:
diff changeset
    23
30496
7cdcc9dd95cb vague cleanup in arith proof tools setup: deleted dead code, more proper structures, clearer arrangement
haftmann
parents: 29302
diff changeset
    24
structure Arith_Data: ARITH_DATA =
9436
62bb04ab4b01 rearranged setup of arithmetic procedures, avoiding global reference values;
wenzelm
parents:
diff changeset
    25
struct
62bb04ab4b01 rearranged setup of arithmetic procedures, avoiding global reference values;
wenzelm
parents:
diff changeset
    26
57952
1a9a6dfc255f updated to named_theorems;
wenzelm
parents: 51717
diff changeset
    27
(* slot for plugging in tactics *)
30686
47a32dd1b86e moved generic arith_tac (formerly silent_arith_tac), verbose_arith_tac (formerly arith_tac) to Arith_Data; simple_arith-tac now named linear_arith_tac
haftmann
parents: 30518
diff changeset
    28
33522
737589bb9bb8 adapted Theory_Data;
wenzelm
parents: 33359
diff changeset
    29
structure Arith_Tactics = Theory_Data
30686
47a32dd1b86e moved generic arith_tac (formerly silent_arith_tac), verbose_arith_tac (formerly arith_tac) to Arith_Data; simple_arith-tac now named linear_arith_tac
haftmann
parents: 30518
diff changeset
    30
(
59657
2441a80fb6c1 eliminated unused arith "verbose" flag -- tools that need options can use the context;
wenzelm
parents: 58820
diff changeset
    31
  type T = (serial * (string * (Proof.context -> int -> tactic))) list;
30686
47a32dd1b86e moved generic arith_tac (formerly silent_arith_tac), verbose_arith_tac (formerly arith_tac) to Arith_Data; simple_arith-tac now named linear_arith_tac
haftmann
parents: 30518
diff changeset
    32
  val empty = [];
33522
737589bb9bb8 adapted Theory_Data;
wenzelm
parents: 33359
diff changeset
    33
  fun merge data : T = AList.merge (op =) (K true) data;
30686
47a32dd1b86e moved generic arith_tac (formerly silent_arith_tac), verbose_arith_tac (formerly arith_tac) to Arith_Data; simple_arith-tac now named linear_arith_tac
haftmann
parents: 30518
diff changeset
    34
);
47a32dd1b86e moved generic arith_tac (formerly silent_arith_tac), verbose_arith_tac (formerly arith_tac) to Arith_Data; simple_arith-tac now named linear_arith_tac
haftmann
parents: 30518
diff changeset
    35
47a32dd1b86e moved generic arith_tac (formerly silent_arith_tac), verbose_arith_tac (formerly arith_tac) to Arith_Data; simple_arith-tac now named linear_arith_tac
haftmann
parents: 30518
diff changeset
    36
fun add_tactic name tac = Arith_Tactics.map (cons (serial (), (name, tac)));
47a32dd1b86e moved generic arith_tac (formerly silent_arith_tac), verbose_arith_tac (formerly arith_tac) to Arith_Data; simple_arith-tac now named linear_arith_tac
haftmann
parents: 30518
diff changeset
    37
59657
2441a80fb6c1 eliminated unused arith "verbose" flag -- tools that need options can use the context;
wenzelm
parents: 58820
diff changeset
    38
fun arith_tac ctxt =
30686
47a32dd1b86e moved generic arith_tac (formerly silent_arith_tac), verbose_arith_tac (formerly arith_tac) to Arith_Data; simple_arith-tac now named linear_arith_tac
haftmann
parents: 30518
diff changeset
    39
  let
42361
23f352990944 modernized structure Proof_Context;
wenzelm
parents: 41539
diff changeset
    40
    val tactics = Arith_Tactics.get (Proof_Context.theory_of ctxt);
59657
2441a80fb6c1 eliminated unused arith "verbose" flag -- tools that need options can use the context;
wenzelm
parents: 58820
diff changeset
    41
    fun invoke (_, (_, tac)) k st = tac ctxt k st;
30686
47a32dd1b86e moved generic arith_tac (formerly silent_arith_tac), verbose_arith_tac (formerly arith_tac) to Arith_Data; simple_arith-tac now named linear_arith_tac
haftmann
parents: 30518
diff changeset
    42
  in FIRST' (map invoke (rev tactics)) end;
47a32dd1b86e moved generic arith_tac (formerly silent_arith_tac), verbose_arith_tac (formerly arith_tac) to Arith_Data; simple_arith-tac now named linear_arith_tac
haftmann
parents: 30518
diff changeset
    43
58820
3ad2759acc52 modernized setup;
wenzelm
parents: 57955
diff changeset
    44
val _ =
3ad2759acc52 modernized setup;
wenzelm
parents: 57955
diff changeset
    45
  Theory.setup
67149
e61557884799 prefer control symbol antiquotations;
wenzelm
parents: 66812
diff changeset
    46
    (Method.setup \<^binding>\<open>arith\<close>
58820
3ad2759acc52 modernized setup;
wenzelm
parents: 57955
diff changeset
    47
      (Scan.succeed (fn ctxt =>
3ad2759acc52 modernized setup;
wenzelm
parents: 57955
diff changeset
    48
        METHOD (fn facts =>
3ad2759acc52 modernized setup;
wenzelm
parents: 57955
diff changeset
    49
          HEADGOAL
67149
e61557884799 prefer control symbol antiquotations;
wenzelm
parents: 66812
diff changeset
    50
            (Method.insert_tac ctxt (rev (Named_Theorems.get ctxt \<^named_theorems>\<open>arith\<close>) @ facts)
61841
4d3527b94f2a more general types Proof.method / context_tactic;
wenzelm
parents: 59657
diff changeset
    51
              THEN' arith_tac ctxt))))
58820
3ad2759acc52 modernized setup;
wenzelm
parents: 57955
diff changeset
    52
      "various arithmetic decision procedures");
30686
47a32dd1b86e moved generic arith_tac (formerly silent_arith_tac), verbose_arith_tac (formerly arith_tac) to Arith_Data; simple_arith-tac now named linear_arith_tac
haftmann
parents: 30518
diff changeset
    53
47a32dd1b86e moved generic arith_tac (formerly silent_arith_tac), verbose_arith_tac (formerly arith_tac) to Arith_Data; simple_arith-tac now named linear_arith_tac
haftmann
parents: 30518
diff changeset
    54
33359
8b673ae1bf39 dedicated theory for loading numeral simprocs
haftmann
parents: 32957
diff changeset
    55
(* some specialized syntactic operations *)
8b673ae1bf39 dedicated theory for loading numeral simprocs
haftmann
parents: 32957
diff changeset
    56
47108
2a1953f0d20d merged fork with new numeral representation (see NEWS)
huffman
parents: 45620
diff changeset
    57
fun mk_number T 1 = HOLogic.numeral_const T $ HOLogic.one_const
2a1953f0d20d merged fork with new numeral representation (see NEWS)
huffman
parents: 45620
diff changeset
    58
  | mk_number T n = HOLogic.mk_number T n;
33359
8b673ae1bf39 dedicated theory for loading numeral simprocs
haftmann
parents: 32957
diff changeset
    59
67149
e61557884799 prefer control symbol antiquotations;
wenzelm
parents: 66812
diff changeset
    60
val mk_plus = HOLogic.mk_binop \<^const_name>\<open>Groups.plus\<close>;
33359
8b673ae1bf39 dedicated theory for loading numeral simprocs
haftmann
parents: 32957
diff changeset
    61
50107
289181e3e524 tuned signature;
wenzelm
parents: 49387
diff changeset
    62
fun mk_minus t =
33359
8b673ae1bf39 dedicated theory for loading numeral simprocs
haftmann
parents: 32957
diff changeset
    63
  let val T = Term.fastype_of t
67149
e61557884799 prefer control symbol antiquotations;
wenzelm
parents: 66812
diff changeset
    64
  in Const (\<^const_name>\<open>Groups.uminus\<close>, T --> T) $ t end;
33359
8b673ae1bf39 dedicated theory for loading numeral simprocs
haftmann
parents: 32957
diff changeset
    65
8b673ae1bf39 dedicated theory for loading numeral simprocs
haftmann
parents: 32957
diff changeset
    66
(*Thus mk_sum[t] yields t+0; longer sums don't have a trailing zero*)
44945
haftmann
parents: 42361
diff changeset
    67
fun mk_sum T [] = mk_number T 0
haftmann
parents: 42361
diff changeset
    68
  | mk_sum T [t, u] = mk_plus (t, u)
33359
8b673ae1bf39 dedicated theory for loading numeral simprocs
haftmann
parents: 32957
diff changeset
    69
  | mk_sum T (t :: ts) = mk_plus (t, mk_sum T ts);
8b673ae1bf39 dedicated theory for loading numeral simprocs
haftmann
parents: 32957
diff changeset
    70
8b673ae1bf39 dedicated theory for loading numeral simprocs
haftmann
parents: 32957
diff changeset
    71
(*this version ALWAYS includes a trailing zero*)
44945
haftmann
parents: 42361
diff changeset
    72
fun long_mk_sum T [] = mk_number T 0
66812
7163b780549d adjusted implementation according to comment
haftmann
parents: 61841
diff changeset
    73
  | long_mk_sum T (t :: ts) = mk_plus (t, long_mk_sum T ts);
33359
8b673ae1bf39 dedicated theory for loading numeral simprocs
haftmann
parents: 32957
diff changeset
    74
8b673ae1bf39 dedicated theory for loading numeral simprocs
haftmann
parents: 32957
diff changeset
    75
(*decompose additions AND subtractions as a sum*)
67149
e61557884799 prefer control symbol antiquotations;
wenzelm
parents: 66812
diff changeset
    76
fun dest_summing (pos, Const (\<^const_name>\<open>Groups.plus\<close>, _) $ t $ u, ts) =
44945
haftmann
parents: 42361
diff changeset
    77
      dest_summing (pos, t, dest_summing (pos, u, ts))
67149
e61557884799 prefer control symbol antiquotations;
wenzelm
parents: 66812
diff changeset
    78
  | dest_summing (pos, Const (\<^const_name>\<open>Groups.minus\<close>, _) $ t $ u, ts) =
44945
haftmann
parents: 42361
diff changeset
    79
      dest_summing (pos, t, dest_summing (not pos, u, ts))
haftmann
parents: 42361
diff changeset
    80
  | dest_summing (pos, t, ts) = (if pos then t else mk_minus t) :: ts;
33359
8b673ae1bf39 dedicated theory for loading numeral simprocs
haftmann
parents: 32957
diff changeset
    81
8b673ae1bf39 dedicated theory for loading numeral simprocs
haftmann
parents: 32957
diff changeset
    82
fun dest_sum t = dest_summing (true, t, []);
8b673ae1bf39 dedicated theory for loading numeral simprocs
haftmann
parents: 32957
diff changeset
    83
8b673ae1bf39 dedicated theory for loading numeral simprocs
haftmann
parents: 32957
diff changeset
    84
30686
47a32dd1b86e moved generic arith_tac (formerly silent_arith_tac), verbose_arith_tac (formerly arith_tac) to Arith_Data; simple_arith-tac now named linear_arith_tac
haftmann
parents: 30518
diff changeset
    85
(* various auxiliary and legacy *)
47a32dd1b86e moved generic arith_tac (formerly silent_arith_tac), verbose_arith_tac (formerly arith_tac) to Arith_Data; simple_arith-tac now named linear_arith_tac
haftmann
parents: 30518
diff changeset
    86
30496
7cdcc9dd95cb vague cleanup in arith proof tools setup: deleted dead code, more proper structures, clearer arrangement
haftmann
parents: 29302
diff changeset
    87
fun prove_conv_nohyps tacs ctxt (t, u) =
7cdcc9dd95cb vague cleanup in arith proof tools setup: deleted dead code, more proper structures, clearer arrangement
haftmann
parents: 29302
diff changeset
    88
  if t aconv u then NONE
7cdcc9dd95cb vague cleanup in arith proof tools setup: deleted dead code, more proper structures, clearer arrangement
haftmann
parents: 29302
diff changeset
    89
  else let val eq = HOLogic.mk_Trueprop (HOLogic.mk_eq (t, u))
7cdcc9dd95cb vague cleanup in arith proof tools setup: deleted dead code, more proper structures, clearer arrangement
haftmann
parents: 29302
diff changeset
    90
  in SOME (Goal.prove ctxt [] [] eq (K (EVERY tacs))) end;
26101
a657683e902a tuned structures in arith_data.ML
haftmann
parents: 25484
diff changeset
    91
30496
7cdcc9dd95cb vague cleanup in arith proof tools setup: deleted dead code, more proper structures, clearer arrangement
haftmann
parents: 29302
diff changeset
    92
fun prove_conv tacs ctxt (_: thm list) = prove_conv_nohyps tacs ctxt;
26101
a657683e902a tuned structures in arith_data.ML
haftmann
parents: 25484
diff changeset
    93
51717
9e7d1c139569 simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents: 50107
diff changeset
    94
fun prove_conv2 expand_tac norm_tac ctxt tu = (* FIXME avoid Drule.export_without_context *)
9e7d1c139569 simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents: 50107
diff changeset
    95
  mk_meta_eq (Drule.export_without_context (Goal.prove ctxt [] []
26101
a657683e902a tuned structures in arith_data.ML
haftmann
parents: 25484
diff changeset
    96
      (HOLogic.mk_Trueprop (HOLogic.mk_eq tu))
51717
9e7d1c139569 simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents: 50107
diff changeset
    97
    (K (EVERY [expand_tac, norm_tac ctxt]))));
26101
a657683e902a tuned structures in arith_data.ML
haftmann
parents: 25484
diff changeset
    98
51717
9e7d1c139569 simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents: 50107
diff changeset
    99
fun simp_all_tac rules ctxt =
9e7d1c139569 simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents: 50107
diff changeset
   100
  ALLGOALS (safe_simp_tac (put_simpset HOL_ss ctxt addsimps rules));
26101
a657683e902a tuned structures in arith_data.ML
haftmann
parents: 25484
diff changeset
   101
51717
9e7d1c139569 simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents: 50107
diff changeset
   102
fun simplify_meta_eq rules ctxt =
9e7d1c139569 simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents: 50107
diff changeset
   103
  simplify (put_simpset HOL_basic_ss ctxt addsimps rules |> Simplifier.add_eqcong @{thm eq_cong2})
9e7d1c139569 simplifier uses proper Proof.context instead of historic type simpset;
wenzelm
parents: 50107
diff changeset
   104
    o mk_meta_eq;
30518
07b45c1aa788 moved some generic nonsense to arith_data.ML
haftmann
parents: 30496
diff changeset
   105
24095
785c3cd7fcb5 moved lin_arith stuff to Tools/lin_arith.ML;
wenzelm
parents: 24076
diff changeset
   106
end;