src/HOL/Import/shuffler.ML
author wenzelm
Mon, 29 Sep 2008 11:46:47 +0200
changeset 28397 389c5e494605
parent 27865 27a8ad9612a3
child 29265 5b4247055bd7
permissions -rw-r--r--
handle _ should be avoided (spurious Interrupt will spoil the game);
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
14620
1be590fd2422 Minor cleanup of headers and some speedup of the HOL4 import.
skalberg
parents: 14518
diff changeset
     1
(*  Title:      HOL/Import/shuffler.ML
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
     2
    ID:         $Id$
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
     3
    Author:     Sebastian Skalberg, TU Muenchen
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
     4
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
     5
Package for proving two terms equal by normalizing (hence the
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
     6
"shuffler" name).  Uses the simplifier for the normalization.
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
     7
*)
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
     8
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
     9
signature Shuffler =
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
    10
sig
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
    11
    val debug      : bool ref
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
    12
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
    13
    val norm_term  : theory -> term -> thm
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
    14
    val make_equal : theory -> term -> term -> thm option
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
    15
    val set_prop   : theory -> term -> (string * thm) list -> (string * thm) option
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
    16
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
    17
    val find_potential: theory -> term -> (string * thm) list
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
    18
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
    19
    val gen_shuffle_tac: theory -> bool -> (string * thm) list -> int -> tactic
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
    20
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
    21
    val shuffle_tac: (string * thm) list -> int -> tactic
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
    22
    val search_tac : (string * thm) list -> int -> tactic
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
    23
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
    24
    val print_shuffles: theory -> unit
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
    25
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
    26
    val add_shuffle_rule: thm -> theory -> theory
18728
6790126ab5f6 simplified type attribute;
wenzelm
parents: 18708
diff changeset
    27
    val shuffle_attr: attribute
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
    28
18708
4b3dadb4fe33 setup: theory -> theory;
wenzelm
parents: 18127
diff changeset
    29
    val setup      : theory -> theory
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
    30
end
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
    31
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
    32
structure Shuffler :> Shuffler =
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
    33
struct
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
    34
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
    35
val debug = ref false
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
    36
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
    37
fun if_debug f x = if !debug then f x else ()
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
    38
val message = if_debug writeln
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
    39
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
    40
(*Prints exceptions readably to users*)
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
    41
fun print_sign_exn_unit sign e =
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
    42
  case e of
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
    43
     THM (msg,i,thms) =>
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
    44
         (writeln ("Exception THM " ^ string_of_int i ^ " raised:\n" ^ msg);
26928
ca87aff1ad2d structure Display: less pervasive operations;
wenzelm
parents: 26690
diff changeset
    45
          List.app Display.print_thm thms)
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
    46
   | THEORY (msg,thys) =>
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
    47
         (writeln ("Exception THEORY raised:\n" ^ msg);
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
    48
          List.app (writeln o Context.str_of_thy) thys)
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
    49
   | TERM (msg,ts) =>
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
    50
         (writeln ("Exception TERM raised:\n" ^ msg);
26939
1035c89b4c02 moved global pretty/string_of functions from Sign to Syntax;
wenzelm
parents: 26928
diff changeset
    51
          List.app (writeln o Syntax.string_of_term_global sign) ts)
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
    52
   | TYPE (msg,Ts,ts) =>
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
    53
         (writeln ("Exception TYPE raised:\n" ^ msg);
26939
1035c89b4c02 moved global pretty/string_of functions from Sign to Syntax;
wenzelm
parents: 26928
diff changeset
    54
          List.app (writeln o Syntax.string_of_typ_global sign) Ts;
1035c89b4c02 moved global pretty/string_of functions from Sign to Syntax;
wenzelm
parents: 26928
diff changeset
    55
          List.app (writeln o Syntax.string_of_term_global sign) ts)
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
    56
   | e => raise e
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
    57
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
    58
(*Prints an exception, then fails*)
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
    59
fun print_sign_exn sign e = (print_sign_exn_unit sign e; raise e)
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
    60
26928
ca87aff1ad2d structure Display: less pervasive operations;
wenzelm
parents: 26690
diff changeset
    61
val string_of_thm = PrintMode.setmp [] Display.string_of_thm;
ca87aff1ad2d structure Display: less pervasive operations;
wenzelm
parents: 26690
diff changeset
    62
val string_of_cterm = PrintMode.setmp [] Display.string_of_cterm;
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
    63
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
    64
fun mk_meta_eq th =
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
    65
    (case concl_of th of
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
    66
         Const("Trueprop",_) $ (Const("op =",_) $ _ $ _) => th RS eq_reflection
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
    67
       | Const("==",_) $ _ $ _ => th
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
    68
       | _ => raise THM("Not an equality",0,[th]))
28397
389c5e494605 handle _ should be avoided (spurious Interrupt will spoil the game);
wenzelm
parents: 27865
diff changeset
    69
    handle _ => raise THM("Couldn't make meta equality",0,[th])  (* FIXME avoid handle _ *)
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
    70
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
    71
fun mk_obj_eq th =
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
    72
    (case concl_of th of
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
    73
         Const("Trueprop",_) $ (Const("op =",_) $ _ $ _) => th
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
    74
       | Const("==",_) $ _ $ _ => th RS meta_eq_to_obj_eq
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
    75
       | _ => raise THM("Not an equality",0,[th]))
28397
389c5e494605 handle _ should be avoided (spurious Interrupt will spoil the game);
wenzelm
parents: 27865
diff changeset
    76
    handle _ => raise THM("Couldn't make object equality",0,[th])  (* FIXME avoid handle _ *)
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
    77
22846
fb79144af9a3 simplified DataFun interfaces;
wenzelm
parents: 22578
diff changeset
    78
structure ShuffleData = TheoryDataFun
fb79144af9a3 simplified DataFun interfaces;
wenzelm
parents: 22578
diff changeset
    79
(
fb79144af9a3 simplified DataFun interfaces;
wenzelm
parents: 22578
diff changeset
    80
  type T = thm list
fb79144af9a3 simplified DataFun interfaces;
wenzelm
parents: 22578
diff changeset
    81
  val empty = []
fb79144af9a3 simplified DataFun interfaces;
wenzelm
parents: 22578
diff changeset
    82
  val copy = I
fb79144af9a3 simplified DataFun interfaces;
wenzelm
parents: 22578
diff changeset
    83
  val extend = I
fb79144af9a3 simplified DataFun interfaces;
wenzelm
parents: 22578
diff changeset
    84
  fun merge _ = Library.gen_union Thm.eq_thm
fb79144af9a3 simplified DataFun interfaces;
wenzelm
parents: 22578
diff changeset
    85
)
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
    86
22846
fb79144af9a3 simplified DataFun interfaces;
wenzelm
parents: 22578
diff changeset
    87
fun print_shuffles thy =
fb79144af9a3 simplified DataFun interfaces;
wenzelm
parents: 22578
diff changeset
    88
  Pretty.writeln (Pretty.big_list "Shuffle theorems:"
fb79144af9a3 simplified DataFun interfaces;
wenzelm
parents: 22578
diff changeset
    89
    (map Display.pretty_thm (ShuffleData.get thy)))
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
    90
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
    91
val weaken =
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
    92
    let
26424
a6cad32a27b0 eliminated theory ProtoPure;
wenzelm
parents: 26277
diff changeset
    93
        val cert = cterm_of Pure.thy
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
    94
        val P = Free("P",propT)
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
    95
        val Q = Free("Q",propT)
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
    96
        val PQ = Logic.mk_implies(P,Q)
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
    97
        val PPQ = Logic.mk_implies(P,PQ)
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
    98
        val cP = cert P
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
    99
        val cQ = cert Q
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   100
        val cPQ = cert PQ
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   101
        val cPPQ = cert PPQ
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   102
        val th1 = assume cPQ |> implies_intr_list [cPQ,cP]
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   103
        val th3 = assume cP
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   104
        val th4 = implies_elim_list (assume cPPQ) [th3,th3]
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   105
                                    |> implies_intr_list [cPPQ,cP]
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   106
    in
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   107
        equal_intr th4 th1 |> standard
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   108
    end
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   109
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   110
val imp_comm =
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   111
    let
26424
a6cad32a27b0 eliminated theory ProtoPure;
wenzelm
parents: 26277
diff changeset
   112
        val cert = cterm_of Pure.thy
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   113
        val P = Free("P",propT)
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   114
        val Q = Free("Q",propT)
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   115
        val R = Free("R",propT)
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   116
        val PQR = Logic.mk_implies(P,Logic.mk_implies(Q,R))
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   117
        val QPR = Logic.mk_implies(Q,Logic.mk_implies(P,R))
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   118
        val cP = cert P
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   119
        val cQ = cert Q
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   120
        val cPQR = cert PQR
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   121
        val cQPR = cert QPR
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   122
        val th1 = implies_elim_list (assume cPQR) [assume cP,assume cQ]
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   123
                                    |> implies_intr_list [cPQR,cQ,cP]
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   124
        val th2 = implies_elim_list (assume cQPR) [assume cQ,assume cP]
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   125
                                    |> implies_intr_list [cQPR,cP,cQ]
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   126
    in
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   127
        equal_intr th1 th2 |> standard
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   128
    end
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   129
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   130
val def_norm =
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   131
    let
26424
a6cad32a27b0 eliminated theory ProtoPure;
wenzelm
parents: 26277
diff changeset
   132
        val cert = cterm_of Pure.thy
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   133
        val aT = TFree("'a",[])
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   134
        val bT = TFree("'b",[])
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   135
        val v = Free("v",aT)
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   136
        val P = Free("P",aT-->bT)
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   137
        val Q = Free("Q",aT-->bT)
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   138
        val cvPQ = cert (list_all ([("v",aT)],Logic.mk_equals(P $ Bound 0,Q $ Bound 0)))
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   139
        val cPQ = cert (Logic.mk_equals(P,Q))
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   140
        val cv = cert v
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   141
        val rew = assume cvPQ
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   142
                         |> forall_elim cv
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   143
                         |> abstract_rule "v" cv
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   144
        val (lhs,rhs) = Logic.dest_equals(concl_of rew)
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   145
        val th1 = transitive (transitive
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   146
                                  (eta_conversion (cert lhs) |> symmetric)
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   147
                                  rew)
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   148
                             (eta_conversion (cert rhs))
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   149
                             |> implies_intr cvPQ
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   150
        val th2 = combination (assume cPQ) (reflexive cv)
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   151
                              |> forall_intr cv
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   152
                              |> implies_intr cPQ
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   153
    in
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   154
        equal_intr th1 th2 |> standard
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   155
    end
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   156
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   157
val all_comm =
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   158
    let
26424
a6cad32a27b0 eliminated theory ProtoPure;
wenzelm
parents: 26277
diff changeset
   159
        val cert = cterm_of Pure.thy
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   160
        val xT = TFree("'a",[])
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   161
        val yT = TFree("'b",[])
27330
1af2598b5f7d Logic.all/mk_equals/mk_implies;
wenzelm
parents: 27173
diff changeset
   162
        val x = Free("x",xT)
1af2598b5f7d Logic.all/mk_equals/mk_implies;
wenzelm
parents: 27173
diff changeset
   163
        val y = Free("y",yT)
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   164
        val P = Free("P",xT-->yT-->propT)
27330
1af2598b5f7d Logic.all/mk_equals/mk_implies;
wenzelm
parents: 27173
diff changeset
   165
        val lhs = Logic.all x (Logic.all y (P $ x $ y))
1af2598b5f7d Logic.all/mk_equals/mk_implies;
wenzelm
parents: 27173
diff changeset
   166
        val rhs = Logic.all y (Logic.all x (P $ x $ y))
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   167
        val cl = cert lhs
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   168
        val cr = cert rhs
27330
1af2598b5f7d Logic.all/mk_equals/mk_implies;
wenzelm
parents: 27173
diff changeset
   169
        val cx = cert x
1af2598b5f7d Logic.all/mk_equals/mk_implies;
wenzelm
parents: 27173
diff changeset
   170
        val cy = cert y
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   171
        val th1 = assume cr
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   172
                         |> forall_elim_list [cy,cx]
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   173
                         |> forall_intr_list [cx,cy]
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   174
                         |> implies_intr cr
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   175
        val th2 = assume cl
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   176
                         |> forall_elim_list [cx,cy]
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   177
                         |> forall_intr_list [cy,cx]
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   178
                         |> implies_intr cl
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   179
    in
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   180
        equal_intr th1 th2 |> standard
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   181
    end
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   182
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   183
val equiv_comm =
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   184
    let
26424
a6cad32a27b0 eliminated theory ProtoPure;
wenzelm
parents: 26277
diff changeset
   185
        val cert = cterm_of Pure.thy
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   186
        val T    = TFree("'a",[])
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   187
        val t    = Free("t",T)
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   188
        val u    = Free("u",T)
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   189
        val ctu  = cert (Logic.mk_equals(t,u))
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   190
        val cut  = cert (Logic.mk_equals(u,t))
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   191
        val th1  = assume ctu |> symmetric |> implies_intr ctu
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   192
        val th2  = assume cut |> symmetric |> implies_intr cut
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   193
    in
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   194
        equal_intr th1 th2 |> standard
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   195
    end
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   196
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   197
(* This simplification procedure rewrites !!x y. P x y
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   198
deterministicly, in order for the normalization function, defined
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   199
below, to handle nested quantifiers robustly *)
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   200
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   201
local
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   202
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   203
exception RESULT of int
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   204
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   205
fun find_bound n (Bound i) = if i = n then raise RESULT 0
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   206
                             else if i = n+1 then raise RESULT 1
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   207
                             else ()
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   208
  | find_bound n (t $ u) = (find_bound n t; find_bound n u)
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   209
  | find_bound n (Abs(_,_,t)) = find_bound (n+1) t
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   210
  | find_bound _ _ = ()
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   211
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   212
fun swap_bound n (Bound i) = if i = n then Bound (n+1)
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   213
                             else if i = n+1 then Bound n
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   214
                             else Bound i
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   215
  | swap_bound n (t $ u) = (swap_bound n t $ swap_bound n u)
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   216
  | swap_bound n (Abs(x,xT,t)) = Abs(x,xT,swap_bound (n+1) t)
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   217
  | swap_bound n t = t
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   218
21078
101aefd61aac slight cleanup
haftmann
parents: 20951
diff changeset
   219
fun rew_th thy (xv as (x,xT)) (yv as (y,yT)) t =
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   220
    let
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   221
        val lhs = list_all ([xv,yv],t)
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   222
        val rhs = list_all ([yv,xv],swap_bound 0 t)
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   223
        val rew = Logic.mk_equals (lhs,rhs)
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   224
        val init = trivial (cterm_of thy rew)
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   225
    in
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   226
        (all_comm RS init handle e => (message "rew_th"; OldGoals.print_exn e))
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   227
    end
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   228
21078
101aefd61aac slight cleanup
haftmann
parents: 20951
diff changeset
   229
fun quant_rewrite thy assumes (t as Const("all",T1) $ (Abs(x,xT,Const("all",T2) $ Abs(y,yT,body)))) =
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   230
    let
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   231
        val res = (find_bound 0 body;2) handle RESULT i => i
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   232
    in
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   233
        case res of
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   234
            0 => SOME (rew_th thy (x,xT) (y,yT) body)
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   235
          | 1 => if string_ord(y,x) = LESS
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   236
                 then
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   237
                     let
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   238
                         val newt = Const("all",T1) $ (Abs(y,xT,Const("all",T2) $ Abs(x,yT,body)))
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   239
                         val t_th    = reflexive (cterm_of thy t)
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   240
                         val newt_th = reflexive (cterm_of thy newt)
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   241
                     in
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   242
                         SOME (transitive t_th newt_th)
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   243
                     end
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   244
                 else NONE
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   245
          | _ => error "norm_term (quant_rewrite) internal error"
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   246
     end
15531
08c8dad8e399 Deleted Library.option type.
skalberg
parents: 14854
diff changeset
   247
  | quant_rewrite _ _ _ = (warning "quant_rewrite: Unknown lhs"; NONE)
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   248
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   249
fun freeze_thaw_term t =
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   250
    let
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   251
        val tvars = term_tvars t
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   252
        val tfree_names = add_term_tfree_names(t,[])
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   253
        val (type_inst,_) =
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   254
            Library.foldl (fn ((inst,used),(w as (v,_),S)) =>
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   255
                      let
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   256
                          val v' = Name.variant used v
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   257
                      in
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   258
                          ((w,TFree(v',S))::inst,v'::used)
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   259
                      end)
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   260
                  (([],tfree_names),tvars)
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   261
        val t' = subst_TVars type_inst t
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   262
    in
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   263
        (t',map (fn (w,TFree(v,S)) => (v,TVar(w,S))
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   264
                  | _ => error "Internal error in Shuffler.freeze_thaw") type_inst)
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   265
    end
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   266
21078
101aefd61aac slight cleanup
haftmann
parents: 20951
diff changeset
   267
fun inst_tfrees thy [] thm = thm
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   268
  | inst_tfrees thy ((name,U)::rest) thm =
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   269
    let
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   270
        val cU = ctyp_of thy U
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   271
        val tfrees = add_term_tfrees (prop_of thm,[])
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   272
        val (rens, thm') = Thm.varifyT'
20951
868120282837 gen_rem(s) abandoned in favour of remove / subtract
haftmann
parents: 20897
diff changeset
   273
    (remove (op = o apsnd fst) name tfrees) thm
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   274
        val mid =
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   275
            case rens of
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   276
                [] => thm'
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   277
              | [((_, S), idx)] => instantiate
21078
101aefd61aac slight cleanup
haftmann
parents: 20951
diff changeset
   278
            ([(ctyp_of thy (TVar (idx, S)), cU)], []) thm'
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   279
              | _ => error "Shuffler.inst_tfrees internal error"
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   280
    in
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   281
        inst_tfrees thy rest mid
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   282
    end
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   283
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   284
fun is_Abs (Abs _) = true
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   285
  | is_Abs _ = false
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   286
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   287
fun eta_redex (t $ Bound 0) =
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   288
    let
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   289
        fun free n (Bound i) = i = n
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   290
          | free n (t $ u) = free n t orelse free n u
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   291
          | free n (Abs(_,_,t)) = free (n+1) t
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   292
          | free n _ = false
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   293
    in
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   294
        not (free 0 t)
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   295
    end
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   296
  | eta_redex _ = false
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   297
21078
101aefd61aac slight cleanup
haftmann
parents: 20951
diff changeset
   298
fun eta_contract thy assumes origt =
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   299
    let
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   300
        val (typet,Tinst) = freeze_thaw_term origt
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   301
        val (init,thaw) = freeze_thaw (reflexive (cterm_of thy typet))
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   302
        val final = inst_tfrees thy Tinst o thaw
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   303
        val t = #1 (Logic.dest_equals (prop_of init))
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   304
        val _ =
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   305
            let
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   306
                val lhs = #1 (Logic.dest_equals (prop_of (final init)))
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   307
            in
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   308
                if not (lhs aconv origt)
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   309
                then (writeln "Something is utterly wrong: (orig,lhs,frozen type,t,tinst)";
26928
ca87aff1ad2d structure Display: less pervasive operations;
wenzelm
parents: 26690
diff changeset
   310
                      writeln (Display.string_of_cterm (cterm_of thy origt));
ca87aff1ad2d structure Display: less pervasive operations;
wenzelm
parents: 26690
diff changeset
   311
                      writeln (Display.string_of_cterm (cterm_of thy lhs));
ca87aff1ad2d structure Display: less pervasive operations;
wenzelm
parents: 26690
diff changeset
   312
                      writeln (Display.string_of_cterm (cterm_of thy typet));
ca87aff1ad2d structure Display: less pervasive operations;
wenzelm
parents: 26690
diff changeset
   313
                      writeln (Display.string_of_cterm (cterm_of thy t));
ca87aff1ad2d structure Display: less pervasive operations;
wenzelm
parents: 26690
diff changeset
   314
                      app (fn (n,T) => writeln (n ^ ": " ^ (Display.string_of_ctyp (ctyp_of thy T)))) Tinst;
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   315
                      writeln "done")
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   316
                else ()
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   317
            end
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   318
    in
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   319
        case t of
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   320
            Const("all",_) $ (Abs(x,xT,Const("==",eqT) $ P $ Q)) =>
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   321
            ((if eta_redex P andalso eta_redex Q
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   322
              then
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   323
                  let
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   324
                      val cert = cterm_of thy
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   325
                      val v = Free(Name.variant (add_term_free_names(t,[])) "v",xT)
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   326
                      val cv = cert v
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   327
                      val ct = cert t
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   328
                      val th = (assume ct)
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   329
                                   |> forall_elim cv
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   330
                                   |> abstract_rule x cv
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   331
                      val ext_th = eta_conversion (cert (Abs(x,xT,P)))
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   332
                      val th' = transitive (symmetric ext_th) th
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   333
                      val cu = cert (prop_of th')
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   334
                      val uth = combination (assume cu) (reflexive cv)
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   335
                      val uth' = (beta_conversion false (cert (Abs(x,xT,Q) $ v)))
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   336
                                     |> transitive uth
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   337
                                     |> forall_intr cv
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   338
                                     |> implies_intr cu
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   339
                      val rew_th = equal_intr (th' |> implies_intr ct) uth'
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   340
                      val res = final rew_th
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   341
                      val lhs = (#1 (Logic.dest_equals (prop_of res)))
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   342
                  in
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   343
                       SOME res
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   344
                  end
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   345
              else NONE)
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   346
             handle e => OldGoals.print_exn e)
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   347
          | _ => NONE
17440
df77edc4f5d0 fixed HOL-light/Isabelle syntax incompatability via more protect_xxx functions
obua
parents: 17188
diff changeset
   348
       end
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   349
21078
101aefd61aac slight cleanup
haftmann
parents: 20951
diff changeset
   350
fun beta_fun thy assume t =
101aefd61aac slight cleanup
haftmann
parents: 20951
diff changeset
   351
    SOME (beta_conversion true (cterm_of thy t))
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   352
17188
a26a4fc323ed Updated import.
obua
parents: 16428
diff changeset
   353
val meta_sym_rew = thm "refl"
a26a4fc323ed Updated import.
obua
parents: 16428
diff changeset
   354
21078
101aefd61aac slight cleanup
haftmann
parents: 20951
diff changeset
   355
fun equals_fun thy assume t =
17188
a26a4fc323ed Updated import.
obua
parents: 16428
diff changeset
   356
    case t of
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   357
        Const("op ==",_) $ u $ v => if Term.term_ord (u,v) = LESS then SOME (meta_sym_rew) else NONE
17188
a26a4fc323ed Updated import.
obua
parents: 16428
diff changeset
   358
      | _ => NONE
a26a4fc323ed Updated import.
obua
parents: 16428
diff changeset
   359
21078
101aefd61aac slight cleanup
haftmann
parents: 20951
diff changeset
   360
fun eta_expand thy assumes origt =
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   361
    let
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   362
        val (typet,Tinst) = freeze_thaw_term origt
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   363
        val (init,thaw) = freeze_thaw (reflexive (cterm_of thy typet))
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   364
        val final = inst_tfrees thy Tinst o thaw
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   365
        val t = #1 (Logic.dest_equals (prop_of init))
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   366
        val _ =
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   367
            let
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   368
                val lhs = #1 (Logic.dest_equals (prop_of (final init)))
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   369
            in
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   370
                if not (lhs aconv origt)
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   371
                then (writeln "Something is utterly wrong: (orig,lhs,frozen type,t,tinst)";
26928
ca87aff1ad2d structure Display: less pervasive operations;
wenzelm
parents: 26690
diff changeset
   372
                      writeln (Display.string_of_cterm (cterm_of thy origt));
ca87aff1ad2d structure Display: less pervasive operations;
wenzelm
parents: 26690
diff changeset
   373
                      writeln (Display.string_of_cterm (cterm_of thy lhs));
ca87aff1ad2d structure Display: less pervasive operations;
wenzelm
parents: 26690
diff changeset
   374
                      writeln (Display.string_of_cterm (cterm_of thy typet));
ca87aff1ad2d structure Display: less pervasive operations;
wenzelm
parents: 26690
diff changeset
   375
                      writeln (Display.string_of_cterm (cterm_of thy t));
ca87aff1ad2d structure Display: less pervasive operations;
wenzelm
parents: 26690
diff changeset
   376
                      app (fn (n,T) => writeln (n ^ ": " ^ (Display.string_of_ctyp (ctyp_of thy T)))) Tinst;
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   377
                      writeln "done")
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   378
                else ()
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   379
            end
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   380
    in
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   381
        case t of
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   382
            Const("==",T) $ P $ Q =>
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   383
            if is_Abs P orelse is_Abs Q
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   384
            then (case domain_type T of
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   385
                      Type("fun",[aT,bT]) =>
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   386
                      let
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   387
                          val cert = cterm_of thy
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   388
                          val vname = Name.variant (add_term_free_names(t,[])) "v"
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   389
                          val v = Free(vname,aT)
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   390
                          val cv = cert v
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   391
                          val ct = cert t
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   392
                          val th1 = (combination (assume ct) (reflexive cv))
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   393
                                        |> forall_intr cv
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   394
                                        |> implies_intr ct
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   395
                          val concl = cert (concl_of th1)
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   396
                          val th2 = (assume concl)
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   397
                                        |> forall_elim cv
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   398
                                        |> abstract_rule vname cv
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   399
                          val (lhs,rhs) = Logic.dest_equals (prop_of th2)
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   400
                          val elhs = eta_conversion (cert lhs)
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   401
                          val erhs = eta_conversion (cert rhs)
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   402
                          val th2' = transitive
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   403
                                         (transitive (symmetric elhs) th2)
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   404
                                         erhs
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   405
                          val res = equal_intr th1 (th2' |> implies_intr concl)
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   406
                          val res' = final res
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   407
                      in
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   408
                          SOME res'
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   409
                      end
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   410
                    | _ => NONE)
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   411
            else NONE
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   412
          | _ => (error ("Bad eta_expand argument" ^ (string_of_cterm (cterm_of thy t))); NONE)
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   413
    end
17959
8db36a108213 OldGoals;
wenzelm
parents: 17892
diff changeset
   414
    handle e => (writeln "eta_expand internal error"; OldGoals.print_exn e)
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   415
14854
61bdf2ae4dc5 removed obsolete sort 'logic';
wenzelm
parents: 14848
diff changeset
   416
fun mk_tfree s = TFree("'"^s,[])
20326
cbf31171c147 fixed generator
obua
parents: 20224
diff changeset
   417
fun mk_free s t = Free (s,t)
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   418
val xT = mk_tfree "a"
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   419
val yT = mk_tfree "b"
27330
1af2598b5f7d Logic.all/mk_equals/mk_implies;
wenzelm
parents: 27173
diff changeset
   420
val x = Free ("x", xT)
1af2598b5f7d Logic.all/mk_equals/mk_implies;
wenzelm
parents: 27173
diff changeset
   421
val y = Free ("y", yT)
20326
cbf31171c147 fixed generator
obua
parents: 20224
diff changeset
   422
val P  = mk_free "P" (xT-->yT-->propT)
cbf31171c147 fixed generator
obua
parents: 20224
diff changeset
   423
val Q  = mk_free "Q" (xT-->yT)
cbf31171c147 fixed generator
obua
parents: 20224
diff changeset
   424
val R  = mk_free "R" (xT-->yT)
cbf31171c147 fixed generator
obua
parents: 20224
diff changeset
   425
val S  = mk_free "S" xT
cbf31171c147 fixed generator
obua
parents: 20224
diff changeset
   426
val S'  = mk_free "S'" xT
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   427
in
21078
101aefd61aac slight cleanup
haftmann
parents: 20951
diff changeset
   428
fun beta_simproc thy = Simplifier.simproc_i
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   429
                      thy
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   430
                      "Beta-contraction"
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   431
                      [Abs("x",xT,Q) $ S]
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   432
                      beta_fun
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   433
21078
101aefd61aac slight cleanup
haftmann
parents: 20951
diff changeset
   434
fun equals_simproc thy = Simplifier.simproc_i
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   435
                      thy
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   436
                      "Ordered rewriting of meta equalities"
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   437
                      [Const("op ==",xT) $ S $ S']
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   438
                      equals_fun
17188
a26a4fc323ed Updated import.
obua
parents: 16428
diff changeset
   439
21078
101aefd61aac slight cleanup
haftmann
parents: 20951
diff changeset
   440
fun quant_simproc thy = Simplifier.simproc_i
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   441
                           thy
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   442
                           "Ordered rewriting of nested quantifiers"
27330
1af2598b5f7d Logic.all/mk_equals/mk_implies;
wenzelm
parents: 27173
diff changeset
   443
                           [Logic.all x (Logic.all y (P $ x $ y))]
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   444
                           quant_rewrite
21078
101aefd61aac slight cleanup
haftmann
parents: 20951
diff changeset
   445
fun eta_expand_simproc thy = Simplifier.simproc_i
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   446
                         thy
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   447
                         "Smart eta-expansion by equivalences"
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   448
                         [Logic.mk_equals(Q,R)]
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   449
                         eta_expand
21078
101aefd61aac slight cleanup
haftmann
parents: 20951
diff changeset
   450
fun eta_contract_simproc thy = Simplifier.simproc_i
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   451
                         thy
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   452
                         "Smart handling of eta-contractions"
27330
1af2598b5f7d Logic.all/mk_equals/mk_implies;
wenzelm
parents: 27173
diff changeset
   453
                         [Logic.all x (Logic.mk_equals (Q $ x, R $ x))]
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   454
                         eta_contract
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   455
end
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   456
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   457
(* Disambiguates the names of bound variables in a term, returning t
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   458
== t' where all the names of bound variables in t' are unique *)
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   459
21078
101aefd61aac slight cleanup
haftmann
parents: 20951
diff changeset
   460
fun disamb_bound thy t =
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   461
    let
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   462
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   463
        fun F (t $ u,idx) =
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   464
            let
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   465
                val (t',idx') = F (t,idx)
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   466
                val (u',idx'') = F (u,idx')
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   467
            in
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   468
                (t' $ u',idx'')
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   469
            end
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   470
          | F (Abs(x,xT,t),idx) =
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   471
            let
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   472
                val x' = "x" ^ (LargeInt.toString idx) (* amazing *)
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   473
                val (t',idx') = F (t,idx+1)
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   474
            in
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   475
                (Abs(x',xT,t'),idx')
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   476
            end
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   477
          | F arg = arg
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   478
        val (t',_) = F (t,0)
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   479
        val ct = cterm_of thy t
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   480
        val ct' = cterm_of thy t'
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   481
        val res = transitive (reflexive ct) (reflexive ct')
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   482
        val _ = message ("disamb_term: " ^ (string_of_thm res))
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   483
    in
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   484
        res
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   485
    end
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   486
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   487
(* Transforms a term t to some normal form t', returning the theorem t
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   488
== t'.  This is originally a help function for make_equal, but might
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   489
be handy in its own right, for example for indexing terms. *)
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   490
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   491
fun norm_term thy t =
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   492
    let
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   493
        val norms = ShuffleData.get thy
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   494
        val ss = Simplifier.theory_context thy empty_ss
17892
62c397c17d18 Simplifier.theory_context;
wenzelm
parents: 17463
diff changeset
   495
          setmksimps single
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   496
          addsimps (map (Thm.transfer thy) norms)
21078
101aefd61aac slight cleanup
haftmann
parents: 20951
diff changeset
   497
          addsimprocs [quant_simproc thy, eta_expand_simproc thy,eta_contract_simproc thy]
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   498
        fun chain f th =
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   499
            let
22902
ac833b4bb7ee moved some Drule operations to Thm (see more_thm.ML);
wenzelm
parents: 22846
diff changeset
   500
                val rhs = Thm.rhs_of th
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   501
            in
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   502
                transitive th (f rhs)
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   503
            end
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   504
        val th =
21078
101aefd61aac slight cleanup
haftmann
parents: 20951
diff changeset
   505
            t |> disamb_bound thy
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   506
              |> chain (Simplifier.full_rewrite ss)
20326
cbf31171c147 fixed generator
obua
parents: 20224
diff changeset
   507
              |> chain eta_conversion
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   508
              |> strip_shyps
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   509
        val _ = message ("norm_term: " ^ (string_of_thm th))
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   510
    in
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   511
        th
17463
e9c1574d0caf removed spurious PolyML.exception_trace;
wenzelm
parents: 17440
diff changeset
   512
    end
21078
101aefd61aac slight cleanup
haftmann
parents: 20951
diff changeset
   513
    handle e => (writeln "norm_term internal error"; print_sign_exn thy e)
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   514
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   515
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   516
(* Closes a theorem with respect to free and schematic variables (does
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   517
not touch type variables, though). *)
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   518
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   519
fun close_thm th =
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   520
    let
22578
b0eb5652f210 removed obsolete sign_of/sign_of_thm;
wenzelm
parents: 21588
diff changeset
   521
        val thy = Thm.theory_of_thm th
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   522
        val c = prop_of th
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   523
        val vars = add_term_frees (c,add_term_vars(c,[]))
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   524
    in
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   525
        Drule.forall_intr_list (map (cterm_of thy) vars) th
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   526
    end
17959
8db36a108213 OldGoals;
wenzelm
parents: 17892
diff changeset
   527
    handle e => (writeln "close_thm internal error"; OldGoals.print_exn e)
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   528
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   529
(* Normalizes a theorem's conclusion using norm_term. *)
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   530
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   531
fun norm_thm thy th =
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   532
    let
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   533
        val c = prop_of th
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   534
    in
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   535
        equal_elim (norm_term thy c) th
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   536
    end
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   537
21078
101aefd61aac slight cleanup
haftmann
parents: 20951
diff changeset
   538
(* make_equal thy t u tries to construct the theorem t == u under the
101aefd61aac slight cleanup
haftmann
parents: 20951
diff changeset
   539
signature thy.  If it succeeds, SOME (t == u) is returned, otherwise
15531
08c8dad8e399 Deleted Library.option type.
skalberg
parents: 14854
diff changeset
   540
NONE is returned. *)
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   541
21078
101aefd61aac slight cleanup
haftmann
parents: 20951
diff changeset
   542
fun make_equal thy t u =
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   543
    let
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   544
        val t_is_t' = norm_term thy t
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   545
        val u_is_u' = norm_term thy u
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   546
        val th = transitive t_is_t' (symmetric u_is_u')
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   547
        val _ = message ("make_equal: SOME " ^ (string_of_thm th))
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   548
    in
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   549
        SOME th
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   550
    end
15531
08c8dad8e399 Deleted Library.option type.
skalberg
parents: 14854
diff changeset
   551
    handle e as THM _ => (message "make_equal: NONE";NONE)
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   552
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   553
fun match_consts ignore t (* th *) =
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   554
    let
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   555
        fun add_consts (Const (c, _), cs) =
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   556
            if c mem_string ignore
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   557
            then cs
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   558
            else insert (op =) c cs
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   559
          | add_consts (t $ u, cs) = add_consts (t, add_consts (u, cs))
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   560
          | add_consts (Abs (_, _, t), cs) = add_consts (t, cs)
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   561
          | add_consts (_, cs) = cs
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   562
        val t_consts = add_consts(t,[])
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   563
    in
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   564
     fn (name,th) =>
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   565
        let
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   566
            val th_consts = add_consts(prop_of th,[])
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   567
        in
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   568
            eq_set(t_consts,th_consts)
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   569
        end
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   570
    end
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   571
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   572
val collect_ignored =
21078
101aefd61aac slight cleanup
haftmann
parents: 20951
diff changeset
   573
    fold_rev (fn thm => fn cs =>
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   574
              let
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   575
                  val (lhs,rhs) = Logic.dest_equals (prop_of thm)
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   576
                  val ignore_lhs = term_consts lhs \\ term_consts rhs
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   577
                  val ignore_rhs = term_consts rhs \\ term_consts lhs
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   578
              in
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   579
                  fold_rev (insert (op =)) cs (ignore_lhs @ ignore_rhs)
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   580
              end)
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   581
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   582
(* set_prop t thms tries to make a theorem with the proposition t from
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   583
one of the theorems thms, by shuffling the propositions around.  If it
15531
08c8dad8e399 Deleted Library.option type.
skalberg
parents: 14854
diff changeset
   584
succeeds, SOME theorem is returned, otherwise NONE.  *)
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   585
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   586
fun set_prop thy t =
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   587
    let
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   588
        val vars = add_term_frees (t,add_term_vars (t,[]))
27330
1af2598b5f7d Logic.all/mk_equals/mk_implies;
wenzelm
parents: 27173
diff changeset
   589
        val closed_t = fold_rev Logic.all vars t
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   590
        val rew_th = norm_term thy closed_t
22902
ac833b4bb7ee moved some Drule operations to Thm (see more_thm.ML);
wenzelm
parents: 22846
diff changeset
   591
        val rhs = Thm.rhs_of rew_th
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   592
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   593
        val shuffles = ShuffleData.get thy
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   594
        fun process [] = NONE
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   595
          | process ((name,th)::thms) =
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   596
            let
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   597
                val norm_th = Thm.varifyT (norm_thm thy (close_thm (Thm.transfer thy th)))
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   598
                val triv_th = trivial rhs
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   599
                val _ = message ("Shuffler.set_prop: Gluing together " ^ (string_of_thm norm_th) ^ " and " ^ (string_of_thm triv_th))
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   600
                val mod_th = case Seq.pull (bicompose false (*true*) (false,norm_th,0) 1 triv_th) of
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   601
                                 SOME(th,_) => SOME th
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   602
                               | NONE => NONE
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   603
            in
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   604
                case mod_th of
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   605
                    SOME mod_th =>
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   606
                    let
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   607
                        val closed_th = equal_elim (symmetric rew_th) mod_th
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   608
                    in
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   609
                        message ("Shuffler.set_prop succeeded by " ^ name);
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   610
                        SOME (name,forall_elim_list (map (cterm_of thy) vars) closed_th)
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   611
                    end
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   612
                  | NONE => process thms
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   613
            end
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   614
            handle e as THM _ => process thms
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   615
    in
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   616
        fn thms =>
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   617
           case process thms of
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   618
               res as SOME (name,th) => if (prop_of th) aconv t
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   619
                                        then res
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   620
                                        else error "Internal error in set_prop"
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   621
             | NONE => NONE
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   622
    end
17959
8db36a108213 OldGoals;
wenzelm
parents: 17892
diff changeset
   623
    handle e => (writeln "set_prop internal error"; OldGoals.print_exn e)
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   624
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   625
fun find_potential thy t =
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   626
    let
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   627
        val shuffles = ShuffleData.get thy
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   628
        val ignored = collect_ignored shuffles []
26662
39483503705f Facts.dest_table;
wenzelm
parents: 26424
diff changeset
   629
        val all_thms =
27865
27a8ad9612a3 moved basic thm operations from structure PureThy to Thm (cf. more_thm.ML);
wenzelm
parents: 27330
diff changeset
   630
          map (`Thm.get_name_hint) (maps #2 (Facts.dest_static [] (PureThy.facts_of thy)))
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   631
    in
26277
461e11226111 removed obsolete PureThy.thms_containing_consts;
wenzelm
parents: 24634
diff changeset
   632
        List.filter (match_consts ignored t) all_thms
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   633
    end
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   634
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   635
fun gen_shuffle_tac thy search thms i st =
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   636
    let
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   637
        val _ = message ("Shuffling " ^ (string_of_thm st))
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   638
        val t = List.nth(prems_of st,i-1)
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   639
        val set = set_prop thy t
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   640
        fun process_tac thms st =
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   641
            case set thms of
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   642
                SOME (_,th) => Seq.of_list (compose (th,i,st))
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   643
              | NONE => Seq.empty
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   644
    in
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   645
        (process_tac thms APPEND (if search
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   646
                                  then process_tac (find_potential thy t)
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   647
                                  else no_tac)) st
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   648
    end
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   649
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   650
fun shuffle_tac thms i st =
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   651
    gen_shuffle_tac (the_context()) false thms i st
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   652
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   653
fun search_tac thms i st =
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   654
    gen_shuffle_tac (the_context()) true thms i st
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   655
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   656
fun shuffle_meth (thms:thm list) ctxt =
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   657
    let
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   658
        val thy = ProofContext.theory_of ctxt
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   659
    in
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   660
        Method.SIMPLE_METHOD' (gen_shuffle_tac thy false (map (pair "") thms))
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   661
    end
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   662
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   663
fun search_meth ctxt =
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   664
    let
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   665
        val thy = ProofContext.theory_of ctxt
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   666
        val prems = Assumption.prems_of ctxt
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   667
    in
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   668
        Method.SIMPLE_METHOD' (gen_shuffle_tac thy true (map (pair "premise") prems))
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   669
    end
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   670
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   671
fun add_shuffle_rule thm thy =
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   672
    let
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   673
        val shuffles = ShuffleData.get thy
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   674
    in
21588
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   675
        if exists (curry Thm.eq_thm thm) shuffles
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   676
        then (warning ((string_of_thm thm) ^ " already known to the shuffler");
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   677
              thy)
cd0dc678a205 simplified method setup;
wenzelm
parents: 21078
diff changeset
   678
        else ShuffleData.put (thm::shuffles) thy
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   679
    end
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   680
20897
3f8d2834b2c4 attribute: Context.mapping;
wenzelm
parents: 20854
diff changeset
   681
val shuffle_attr = Thm.declaration_attribute (fn th => Context.mapping (add_shuffle_rule th) I);
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   682
18708
4b3dadb4fe33 setup: theory -> theory;
wenzelm
parents: 18127
diff changeset
   683
val setup =
22846
fb79144af9a3 simplified DataFun interfaces;
wenzelm
parents: 22578
diff changeset
   684
  Method.add_method ("shuffle_tac",
fb79144af9a3 simplified DataFun interfaces;
wenzelm
parents: 22578
diff changeset
   685
    Method.thms_ctxt_args shuffle_meth,"solve goal by shuffling terms around") #>
fb79144af9a3 simplified DataFun interfaces;
wenzelm
parents: 22578
diff changeset
   686
  Method.add_method ("search_tac",
fb79144af9a3 simplified DataFun interfaces;
wenzelm
parents: 22578
diff changeset
   687
    Method.ctxt_args search_meth,"search for suitable theorems") #>
18708
4b3dadb4fe33 setup: theory -> theory;
wenzelm
parents: 18127
diff changeset
   688
  add_shuffle_rule weaken #>
4b3dadb4fe33 setup: theory -> theory;
wenzelm
parents: 18127
diff changeset
   689
  add_shuffle_rule equiv_comm #>
4b3dadb4fe33 setup: theory -> theory;
wenzelm
parents: 18127
diff changeset
   690
  add_shuffle_rule imp_comm #>
4b3dadb4fe33 setup: theory -> theory;
wenzelm
parents: 18127
diff changeset
   691
  add_shuffle_rule Drule.norm_hhf_eq #>
4b3dadb4fe33 setup: theory -> theory;
wenzelm
parents: 18127
diff changeset
   692
  add_shuffle_rule Drule.triv_forall_equality #>
18728
6790126ab5f6 simplified type attribute;
wenzelm
parents: 18708
diff changeset
   693
  Attrib.add_attributes [("shuffle_rule", Attrib.no_args shuffle_attr, "declare rule for shuffler")]
18708
4b3dadb4fe33 setup: theory -> theory;
wenzelm
parents: 18127
diff changeset
   694
14516
a183dec876ab Added HOL proof importer.
skalberg
parents:
diff changeset
   695
end