src/HOL/Tools/transfer.ML
author wenzelm
Mon, 05 Aug 2013 15:03:52 +0200
changeset 52861 e93d73b51fd0
parent 52358 f4c4bcb0d564
child 52883 0a7c97c76f46
permissions -rw-r--r--
commands with overlay remain visible, to avoid loosing printed output;
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
47325
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
     1
(*  Title:      HOL/Tools/transfer.ML
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
     2
    Author:     Brian Huffman, TU Muenchen
51956
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
     3
    Author:     Ondrej Kuncar, TU Muenchen
47325
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
     4
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
     5
Generic theorem transfer method.
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
     6
*)
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
     7
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
     8
signature TRANSFER =
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
     9
sig
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
    10
  val prep_conv: conv
51956
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
    11
  val get_transfer_raw: Proof.context -> thm list
47503
cb44d09d9d22 add theory data for relator identity rules;
huffman
parents: 47356
diff changeset
    12
  val get_relator_eq: Proof.context -> thm list
49625
06cf80661e7a new get function for non-symmetric relator_eq & tuned
kuncar
parents: 48066
diff changeset
    13
  val get_sym_relator_eq: Proof.context -> thm list
51954
2e3f9e72b8c4 publish a private function
kuncar
parents: 51437
diff changeset
    14
  val get_relator_eq_raw: Proof.context -> thm list
51956
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
    15
  val get_relator_domain: Proof.context -> thm list
47325
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
    16
  val transfer_add: attribute
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
    17
  val transfer_del: attribute
52354
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
    18
  val transferred_attribute: thm list -> attribute
52358
f4c4bcb0d564 implement 'untransferred' attribute, which is like 'transferred' but works in the opposite direction
huffman
parents: 52354
diff changeset
    19
  val untransferred_attribute: thm list -> attribute
51956
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
    20
  val transfer_domain_add: attribute
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
    21
  val transfer_domain_del: attribute
52354
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
    22
  val transfer_rule_of_term: Proof.context -> bool -> term -> thm
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
    23
  val transfer_rule_of_lhs: Proof.context -> term -> thm
47658
7631f6f7873d enable variant of transfer method that proves an implication instead of an equivalence
huffman
parents: 47635
diff changeset
    24
  val transfer_tac: bool -> Proof.context -> int -> tactic
47635
ebb79474262c rename 'correspondence' method to 'transfer_prover'
huffman
parents: 47618
diff changeset
    25
  val transfer_prover_tac: Proof.context -> int -> tactic
52354
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
    26
  val gen_frees_tac: (string * typ) list -> Proof.context -> int -> tactic
47325
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
    27
  val setup: theory -> theory
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
    28
end
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
    29
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
    30
structure Transfer : TRANSFER =
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
    31
struct
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
    32
48064
7bd9e18ce058 unify theory-data structures for transfer package
huffman
parents: 47803
diff changeset
    33
(** Theory Data **)
7bd9e18ce058 unify theory-data structures for transfer package
huffman
parents: 47803
diff changeset
    34
7bd9e18ce058 unify theory-data structures for transfer package
huffman
parents: 47803
diff changeset
    35
structure Data = Generic_Data
47325
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
    36
(
48064
7bd9e18ce058 unify theory-data structures for transfer package
huffman
parents: 47803
diff changeset
    37
  type T =
7bd9e18ce058 unify theory-data structures for transfer package
huffman
parents: 47803
diff changeset
    38
    { transfer_raw : thm Item_Net.T,
48065
8aa05d38299a transfer method now avoids generalizing over free variables that are known to appear in registered transfer rules
huffman
parents: 48064
diff changeset
    39
      known_frees : (string * typ) list,
52354
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
    40
      compound_lhs : unit Net.net,
48066
c6783c9b87bf transfer method now handles transfer rules for compound terms, e.g. locale-defined constants with hidden parameters
huffman
parents: 48065
diff changeset
    41
      compound_rhs : unit Net.net,
51437
8739f8abbecb fixing transfer tactic - unfold fully identity relation by using relator_eq
kuncar
parents: 51374
diff changeset
    42
      relator_eq : thm Item_Net.T,
51956
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
    43
      relator_eq_raw : thm Item_Net.T,
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
    44
      relator_domain : thm Item_Net.T }
48064
7bd9e18ce058 unify theory-data structures for transfer package
huffman
parents: 47803
diff changeset
    45
  val empty =
52354
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
    46
    { transfer_raw = Thm.intro_rules,
48065
8aa05d38299a transfer method now avoids generalizing over free variables that are known to appear in registered transfer rules
huffman
parents: 48064
diff changeset
    47
      known_frees = [],
52354
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
    48
      compound_lhs = Net.empty,
48066
c6783c9b87bf transfer method now handles transfer rules for compound terms, e.g. locale-defined constants with hidden parameters
huffman
parents: 48065
diff changeset
    49
      compound_rhs = Net.empty,
51437
8739f8abbecb fixing transfer tactic - unfold fully identity relation by using relator_eq
kuncar
parents: 51374
diff changeset
    50
      relator_eq = Thm.full_rules,
51956
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
    51
      relator_eq_raw = Thm.full_rules,
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
    52
      relator_domain = Thm.full_rules }
48064
7bd9e18ce058 unify theory-data structures for transfer package
huffman
parents: 47803
diff changeset
    53
  val extend = I
48066
c6783c9b87bf transfer method now handles transfer rules for compound terms, e.g. locale-defined constants with hidden parameters
huffman
parents: 48065
diff changeset
    54
  fun merge
c6783c9b87bf transfer method now handles transfer rules for compound terms, e.g. locale-defined constants with hidden parameters
huffman
parents: 48065
diff changeset
    55
    ( { transfer_raw = t1, known_frees = k1,
52354
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
    56
        compound_lhs = l1,
51437
8739f8abbecb fixing transfer tactic - unfold fully identity relation by using relator_eq
kuncar
parents: 51374
diff changeset
    57
        compound_rhs = c1, relator_eq = r1,
51956
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
    58
        relator_eq_raw = rw1, relator_domain = rd1 },
48066
c6783c9b87bf transfer method now handles transfer rules for compound terms, e.g. locale-defined constants with hidden parameters
huffman
parents: 48065
diff changeset
    59
      { transfer_raw = t2, known_frees = k2,
52354
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
    60
        compound_lhs = l2,
51437
8739f8abbecb fixing transfer tactic - unfold fully identity relation by using relator_eq
kuncar
parents: 51374
diff changeset
    61
        compound_rhs = c2, relator_eq = r2,
51956
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
    62
        relator_eq_raw = rw2, relator_domain = rd2 } ) =
48064
7bd9e18ce058 unify theory-data structures for transfer package
huffman
parents: 47803
diff changeset
    63
    { transfer_raw = Item_Net.merge (t1, t2),
48065
8aa05d38299a transfer method now avoids generalizing over free variables that are known to appear in registered transfer rules
huffman
parents: 48064
diff changeset
    64
      known_frees = Library.merge (op =) (k1, k2),
52354
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
    65
      compound_lhs = Net.merge (K true) (l1, l2),
48066
c6783c9b87bf transfer method now handles transfer rules for compound terms, e.g. locale-defined constants with hidden parameters
huffman
parents: 48065
diff changeset
    66
      compound_rhs = Net.merge (K true) (c1, c2),
51437
8739f8abbecb fixing transfer tactic - unfold fully identity relation by using relator_eq
kuncar
parents: 51374
diff changeset
    67
      relator_eq = Item_Net.merge (r1, r2),
51956
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
    68
      relator_eq_raw = Item_Net.merge (rw1, rw2),
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
    69
      relator_domain = Item_Net.merge (rd1, rd2) }
47325
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
    70
)
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
    71
51956
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
    72
fun get_transfer_raw ctxt = ctxt
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
    73
  |> (Item_Net.content o #transfer_raw o Data.get o Context.Proof)
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
    74
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
    75
fun get_known_frees ctxt = ctxt
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
    76
  |> (#known_frees o Data.get o Context.Proof)
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
    77
52354
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
    78
fun get_compound_lhs ctxt = ctxt
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
    79
  |> (#compound_lhs o Data.get o Context.Proof)
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
    80
51956
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
    81
fun get_compound_rhs ctxt = ctxt
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
    82
  |> (#compound_rhs o Data.get o Context.Proof)
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
    83
48064
7bd9e18ce058 unify theory-data structures for transfer package
huffman
parents: 47803
diff changeset
    84
fun get_relator_eq ctxt = ctxt
7bd9e18ce058 unify theory-data structures for transfer package
huffman
parents: 47803
diff changeset
    85
  |> (Item_Net.content o #relator_eq o Data.get o Context.Proof)
49625
06cf80661e7a new get function for non-symmetric relator_eq & tuned
kuncar
parents: 48066
diff changeset
    86
  |> map safe_mk_meta_eq
06cf80661e7a new get function for non-symmetric relator_eq & tuned
kuncar
parents: 48066
diff changeset
    87
06cf80661e7a new get function for non-symmetric relator_eq & tuned
kuncar
parents: 48066
diff changeset
    88
fun get_sym_relator_eq ctxt = ctxt
06cf80661e7a new get function for non-symmetric relator_eq & tuned
kuncar
parents: 48066
diff changeset
    89
  |> (Item_Net.content o #relator_eq o Data.get o Context.Proof)
06cf80661e7a new get function for non-symmetric relator_eq & tuned
kuncar
parents: 48066
diff changeset
    90
  |> map (Thm.symmetric o safe_mk_meta_eq)
48064
7bd9e18ce058 unify theory-data structures for transfer package
huffman
parents: 47803
diff changeset
    91
51437
8739f8abbecb fixing transfer tactic - unfold fully identity relation by using relator_eq
kuncar
parents: 51374
diff changeset
    92
fun get_relator_eq_raw ctxt = ctxt
8739f8abbecb fixing transfer tactic - unfold fully identity relation by using relator_eq
kuncar
parents: 51374
diff changeset
    93
  |> (Item_Net.content o #relator_eq_raw o Data.get o Context.Proof)
8739f8abbecb fixing transfer tactic - unfold fully identity relation by using relator_eq
kuncar
parents: 51374
diff changeset
    94
51956
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
    95
fun get_relator_domain ctxt = ctxt
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
    96
  |> (Item_Net.content o #relator_domain o Data.get o Context.Proof)
48065
8aa05d38299a transfer method now avoids generalizing over free variables that are known to appear in registered transfer rules
huffman
parents: 48064
diff changeset
    97
52354
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
    98
fun map_data f1 f2 f3 f4 f5 f6 f7
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
    99
  { transfer_raw, known_frees, compound_lhs, compound_rhs,
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   100
    relator_eq, relator_eq_raw, relator_domain } =
48065
8aa05d38299a transfer method now avoids generalizing over free variables that are known to appear in registered transfer rules
huffman
parents: 48064
diff changeset
   101
  { transfer_raw = f1 transfer_raw,
8aa05d38299a transfer method now avoids generalizing over free variables that are known to appear in registered transfer rules
huffman
parents: 48064
diff changeset
   102
    known_frees = f2 known_frees,
52354
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   103
    compound_lhs = f3 compound_lhs,
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   104
    compound_rhs = f4 compound_rhs,
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   105
    relator_eq = f5 relator_eq,
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   106
    relator_eq_raw = f6 relator_eq_raw,
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   107
    relator_domain = f7 relator_domain }
48064
7bd9e18ce058 unify theory-data structures for transfer package
huffman
parents: 47803
diff changeset
   108
52354
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   109
fun map_transfer_raw   f = map_data f I I I I I I
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   110
fun map_known_frees    f = map_data I f I I I I I
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   111
fun map_compound_lhs   f = map_data I I f I I I I
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   112
fun map_compound_rhs   f = map_data I I I f I I I
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   113
fun map_relator_eq     f = map_data I I I I f I I
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   114
fun map_relator_eq_raw f = map_data I I I I I f I
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   115
fun map_relator_domain f = map_data I I I I I I f
47503
cb44d09d9d22 add theory data for relator identity rules;
huffman
parents: 47356
diff changeset
   116
48065
8aa05d38299a transfer method now avoids generalizing over free variables that are known to appear in registered transfer rules
huffman
parents: 48064
diff changeset
   117
fun add_transfer_thm thm = Data.map
8aa05d38299a transfer method now avoids generalizing over free variables that are known to appear in registered transfer rules
huffman
parents: 48064
diff changeset
   118
  (map_transfer_raw (Item_Net.update thm) o
52354
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   119
   map_compound_lhs
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   120
     (case HOLogic.dest_Trueprop (Thm.concl_of thm) of
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   121
        Const (@{const_name Rel}, _) $ _ $ (lhs as (_ $ _)) $ _ =>
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   122
          Net.insert_term_safe (K true) (lhs, ())
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   123
      | _ => I) o
48066
c6783c9b87bf transfer method now handles transfer rules for compound terms, e.g. locale-defined constants with hidden parameters
huffman
parents: 48065
diff changeset
   124
   map_compound_rhs
c6783c9b87bf transfer method now handles transfer rules for compound terms, e.g. locale-defined constants with hidden parameters
huffman
parents: 48065
diff changeset
   125
     (case HOLogic.dest_Trueprop (Thm.concl_of thm) of
52354
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   126
        Const (@{const_name Rel}, _) $ _ $ _ $ (rhs as (_ $ _)) =>
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   127
          Net.insert_term_safe (K true) (rhs, ())
48066
c6783c9b87bf transfer method now handles transfer rules for compound terms, e.g. locale-defined constants with hidden parameters
huffman
parents: 48065
diff changeset
   128
      | _ => I) o
48065
8aa05d38299a transfer method now avoids generalizing over free variables that are known to appear in registered transfer rules
huffman
parents: 48064
diff changeset
   129
   map_known_frees (Term.add_frees (Thm.concl_of thm)))
8aa05d38299a transfer method now avoids generalizing over free variables that are known to appear in registered transfer rules
huffman
parents: 48064
diff changeset
   130
48064
7bd9e18ce058 unify theory-data structures for transfer package
huffman
parents: 47803
diff changeset
   131
fun del_transfer_thm thm = Data.map (map_transfer_raw (Item_Net.remove thm))
7bd9e18ce058 unify theory-data structures for transfer package
huffman
parents: 47803
diff changeset
   132
47325
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
   133
(** Conversions **)
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
   134
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
   135
val Rel_rule = Thm.symmetric @{thm Rel_def}
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
   136
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
   137
fun dest_funcT cT =
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
   138
  (case Thm.dest_ctyp cT of [T, U] => (T, U)
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
   139
    | _ => raise TYPE ("dest_funcT", [Thm.typ_of cT], []))
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
   140
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
   141
fun Rel_conv ct =
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
   142
  let val (cT, cT') = dest_funcT (Thm.ctyp_of_term ct)
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
   143
      val (cU, _) = dest_funcT cT'
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
   144
  in Drule.instantiate' [SOME cT, SOME cU] [SOME ct] Rel_rule end
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
   145
47635
ebb79474262c rename 'correspondence' method to 'transfer_prover'
huffman
parents: 47618
diff changeset
   146
(* Conversion to preprocess a transfer rule *)
51955
04d9381bebff try to detect assumptions of transfer rules that are in a shape of a transfer rule
kuncar
parents: 51954
diff changeset
   147
fun safe_Rel_conv ct =
51956
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   148
  Conv.try_conv (HOLogic.Trueprop_conv (Conv.fun_conv (Conv.fun_conv Rel_conv))) ct
51955
04d9381bebff try to detect assumptions of transfer rules that are in a shape of a transfer rule
kuncar
parents: 51954
diff changeset
   149
47325
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
   150
fun prep_conv ct = (
51955
04d9381bebff try to detect assumptions of transfer rules that are in a shape of a transfer rule
kuncar
parents: 51954
diff changeset
   151
      Conv.implies_conv safe_Rel_conv prep_conv
47325
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
   152
      else_conv
51955
04d9381bebff try to detect assumptions of transfer rules that are in a shape of a transfer rule
kuncar
parents: 51954
diff changeset
   153
      safe_Rel_conv
47325
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
   154
      else_conv
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
   155
      Conv.all_conv) ct
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
   156
49975
faf4afed009f transfer package: more flexible handling of equality relations using is_equality predicate
huffman
parents: 49625
diff changeset
   157
(** Replacing explicit equalities with is_equality premises **)
faf4afed009f transfer package: more flexible handling of equality relations using is_equality predicate
huffman
parents: 49625
diff changeset
   158
faf4afed009f transfer package: more flexible handling of equality relations using is_equality predicate
huffman
parents: 49625
diff changeset
   159
fun mk_is_equality t =
faf4afed009f transfer package: more flexible handling of equality relations using is_equality predicate
huffman
parents: 49625
diff changeset
   160
  Const (@{const_name is_equality}, Term.fastype_of t --> HOLogic.boolT) $ t
47325
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
   161
49975
faf4afed009f transfer package: more flexible handling of equality relations using is_equality predicate
huffman
parents: 49625
diff changeset
   162
val is_equality_lemma =
faf4afed009f transfer package: more flexible handling of equality relations using is_equality predicate
huffman
parents: 49625
diff changeset
   163
  @{lemma "(!!R. is_equality R ==> PROP (P R)) == PROP (P (op =))"
faf4afed009f transfer package: more flexible handling of equality relations using is_equality predicate
huffman
parents: 49625
diff changeset
   164
    by (unfold is_equality_def, rule, drule meta_spec,
faf4afed009f transfer package: more flexible handling of equality relations using is_equality predicate
huffman
parents: 49625
diff changeset
   165
      erule meta_mp, rule refl, simp)}
47325
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
   166
49975
faf4afed009f transfer package: more flexible handling of equality relations using is_equality predicate
huffman
parents: 49625
diff changeset
   167
fun gen_abstract_equalities (dest : term -> term * (term -> term)) thm =
47325
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
   168
  let
49975
faf4afed009f transfer package: more flexible handling of equality relations using is_equality predicate
huffman
parents: 49625
diff changeset
   169
    val thy = Thm.theory_of_thm thm
faf4afed009f transfer package: more flexible handling of equality relations using is_equality predicate
huffman
parents: 49625
diff changeset
   170
    val prop = Thm.prop_of thm
faf4afed009f transfer package: more flexible handling of equality relations using is_equality predicate
huffman
parents: 49625
diff changeset
   171
    val (t, mk_prop') = dest prop
52354
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   172
    (* Only consider "op =" at non-base types *)
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   173
    fun is_eq (Const (@{const_name HOL.eq}, Type ("fun", [T, _]))) =
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   174
        (case T of Type (_, []) => false | _ => true)
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   175
      | is_eq _ = false
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   176
    val add_eqs = Term.fold_aterms (fn t => if is_eq t then insert (op =) t else I)
49975
faf4afed009f transfer package: more flexible handling of equality relations using is_equality predicate
huffman
parents: 49625
diff changeset
   177
    val eq_consts = rev (add_eqs t [])
faf4afed009f transfer package: more flexible handling of equality relations using is_equality predicate
huffman
parents: 49625
diff changeset
   178
    val eqTs = map (snd o dest_Const) eq_consts
faf4afed009f transfer package: more flexible handling of equality relations using is_equality predicate
huffman
parents: 49625
diff changeset
   179
    val used = Term.add_free_names prop []
faf4afed009f transfer package: more flexible handling of equality relations using is_equality predicate
huffman
parents: 49625
diff changeset
   180
    val names = map (K "") eqTs |> Name.variant_list used
faf4afed009f transfer package: more flexible handling of equality relations using is_equality predicate
huffman
parents: 49625
diff changeset
   181
    val frees = map Free (names ~~ eqTs)
faf4afed009f transfer package: more flexible handling of equality relations using is_equality predicate
huffman
parents: 49625
diff changeset
   182
    val prems = map (HOLogic.mk_Trueprop o mk_is_equality) frees
faf4afed009f transfer package: more flexible handling of equality relations using is_equality predicate
huffman
parents: 49625
diff changeset
   183
    val prop1 = mk_prop' (Term.subst_atomic (eq_consts ~~ frees) t)
faf4afed009f transfer package: more flexible handling of equality relations using is_equality predicate
huffman
parents: 49625
diff changeset
   184
    val prop2 = fold Logic.all frees (Logic.list_implies (prems, prop1))
faf4afed009f transfer package: more flexible handling of equality relations using is_equality predicate
huffman
parents: 49625
diff changeset
   185
    val cprop = Thm.cterm_of thy prop2
faf4afed009f transfer package: more flexible handling of equality relations using is_equality predicate
huffman
parents: 49625
diff changeset
   186
    val equal_thm = Raw_Simplifier.rewrite false [is_equality_lemma] cprop
faf4afed009f transfer package: more flexible handling of equality relations using is_equality predicate
huffman
parents: 49625
diff changeset
   187
    fun forall_elim thm = Thm.forall_elim_vars (Thm.maxidx_of thm + 1) thm
47325
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
   188
  in
49975
faf4afed009f transfer package: more flexible handling of equality relations using is_equality predicate
huffman
parents: 49625
diff changeset
   189
    forall_elim (thm COMP (equal_thm COMP @{thm equal_elim_rule2}))
faf4afed009f transfer package: more flexible handling of equality relations using is_equality predicate
huffman
parents: 49625
diff changeset
   190
  end
faf4afed009f transfer package: more flexible handling of equality relations using is_equality predicate
huffman
parents: 49625
diff changeset
   191
    handle TERM _ => thm
faf4afed009f transfer package: more flexible handling of equality relations using is_equality predicate
huffman
parents: 49625
diff changeset
   192
faf4afed009f transfer package: more flexible handling of equality relations using is_equality predicate
huffman
parents: 49625
diff changeset
   193
fun abstract_equalities_transfer thm =
faf4afed009f transfer package: more flexible handling of equality relations using is_equality predicate
huffman
parents: 49625
diff changeset
   194
  let
faf4afed009f transfer package: more flexible handling of equality relations using is_equality predicate
huffman
parents: 49625
diff changeset
   195
    fun dest prop =
faf4afed009f transfer package: more flexible handling of equality relations using is_equality predicate
huffman
parents: 49625
diff changeset
   196
      let
faf4afed009f transfer package: more flexible handling of equality relations using is_equality predicate
huffman
parents: 49625
diff changeset
   197
        val prems = Logic.strip_imp_prems prop
faf4afed009f transfer package: more flexible handling of equality relations using is_equality predicate
huffman
parents: 49625
diff changeset
   198
        val concl = HOLogic.dest_Trueprop (Logic.strip_imp_concl prop)
faf4afed009f transfer package: more flexible handling of equality relations using is_equality predicate
huffman
parents: 49625
diff changeset
   199
        val ((rel, x), y) = apfst Term.dest_comb (Term.dest_comb concl)
faf4afed009f transfer package: more flexible handling of equality relations using is_equality predicate
huffman
parents: 49625
diff changeset
   200
      in
faf4afed009f transfer package: more flexible handling of equality relations using is_equality predicate
huffman
parents: 49625
diff changeset
   201
        (rel, fn rel' =>
faf4afed009f transfer package: more flexible handling of equality relations using is_equality predicate
huffman
parents: 49625
diff changeset
   202
          Logic.list_implies (prems, HOLogic.mk_Trueprop (rel' $ x $ y)))
faf4afed009f transfer package: more flexible handling of equality relations using is_equality predicate
huffman
parents: 49625
diff changeset
   203
      end
faf4afed009f transfer package: more flexible handling of equality relations using is_equality predicate
huffman
parents: 49625
diff changeset
   204
  in
faf4afed009f transfer package: more flexible handling of equality relations using is_equality predicate
huffman
parents: 49625
diff changeset
   205
    gen_abstract_equalities dest thm
faf4afed009f transfer package: more flexible handling of equality relations using is_equality predicate
huffman
parents: 49625
diff changeset
   206
  end
faf4afed009f transfer package: more flexible handling of equality relations using is_equality predicate
huffman
parents: 49625
diff changeset
   207
faf4afed009f transfer package: more flexible handling of equality relations using is_equality predicate
huffman
parents: 49625
diff changeset
   208
fun abstract_equalities_relator_eq rel_eq_thm =
faf4afed009f transfer package: more flexible handling of equality relations using is_equality predicate
huffman
parents: 49625
diff changeset
   209
  gen_abstract_equalities (fn x => (x, I))
faf4afed009f transfer package: more flexible handling of equality relations using is_equality predicate
huffman
parents: 49625
diff changeset
   210
    (rel_eq_thm RS @{thm is_equality_def [THEN iffD2]})
faf4afed009f transfer package: more flexible handling of equality relations using is_equality predicate
huffman
parents: 49625
diff changeset
   211
51956
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   212
fun abstract_equalities_domain thm =
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   213
  let
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   214
    fun dest prop =
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   215
      let
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   216
        val prems = Logic.strip_imp_prems prop
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   217
        val concl = HOLogic.dest_Trueprop (Logic.strip_imp_concl prop)
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   218
        val ((dom, x), y) = apfst Term.dest_comb (Term.dest_comb concl)
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   219
      in
51996
26aecb553c74 abstract equalities only in a correspondence relation in a transfer domain rule
kuncar
parents: 51956
diff changeset
   220
        (x, fn x' => Logic.list_implies (prems, HOLogic.mk_Trueprop (dom $ x' $ y)))
51956
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   221
      end
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   222
  in
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   223
    gen_abstract_equalities dest thm
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   224
  end 
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   225
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   226
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   227
(** Replacing explicit Domainp predicates with Domainp assumptions **)
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   228
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   229
fun mk_Domainp_assm (T, R) =
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   230
  HOLogic.mk_eq ((Const (@{const_name Domainp}, Term.fastype_of T --> Term.fastype_of R) $ T), R)
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   231
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   232
val Domainp_lemma =
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   233
  @{lemma "(!!R. Domainp T = R ==> PROP (P R)) == PROP (P (Domainp T))"
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   234
    by (rule, drule meta_spec,
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   235
      erule meta_mp, rule refl, simp)}
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   236
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   237
fun fold_Domainp f (t as Const (@{const_name Domainp},_) $ (Var (_,_))) = f t
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   238
  | fold_Domainp f (t $ u) = fold_Domainp f t #> fold_Domainp f u
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   239
  | fold_Domainp f (Abs (_, _, t)) = fold_Domainp f t
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   240
  | fold_Domainp _ _ = I
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   241
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   242
fun subst_terms tab t = 
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   243
  let
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   244
    val t' = Termtab.lookup tab t
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   245
  in
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   246
    case t' of
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   247
      SOME t' => t'
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   248
      | NONE => 
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   249
        (case t of
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   250
          u $ v => (subst_terms tab u) $ (subst_terms tab v)
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   251
          | Abs (a, T, t) => Abs (a, T, subst_terms tab t)
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   252
          | t => t)
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   253
  end
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   254
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   255
fun gen_abstract_domains (dest : term -> term * (term -> term)) thm =
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   256
  let
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   257
    val thy = Thm.theory_of_thm thm
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   258
    val prop = Thm.prop_of thm
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   259
    val (t, mk_prop') = dest prop
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   260
    val Domainp_tms = rev (fold_Domainp (fn t => insert op= t) t [])
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   261
    val Domainp_Ts = map (snd o dest_funT o snd o dest_Const o fst o dest_comb) Domainp_tms
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   262
    val used = Term.add_free_names t []
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   263
    val rels = map (snd o dest_comb) Domainp_tms
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   264
    val rel_names = map (fst o fst o dest_Var) rels
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   265
    val names = map (fn name => ("D" ^ name)) rel_names |> Name.variant_list used
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   266
    val frees = map Free (names ~~ Domainp_Ts)
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   267
    val prems = map (HOLogic.mk_Trueprop o mk_Domainp_assm) (rels ~~ frees);
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   268
    val t' = subst_terms (fold Termtab.update (Domainp_tms ~~ frees) Termtab.empty) t
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   269
    val prop1 = fold Logic.all frees (Logic.list_implies (prems, mk_prop' t'))
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   270
    val prop2 = Logic.list_rename_params (rev names) prop1
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   271
    val cprop = Thm.cterm_of thy prop2
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   272
    val equal_thm = Raw_Simplifier.rewrite false [Domainp_lemma] cprop
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   273
    fun forall_elim thm = Thm.forall_elim_vars (Thm.maxidx_of thm + 1) thm;
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   274
  in
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   275
    forall_elim (thm COMP (equal_thm COMP @{thm equal_elim_rule2}))
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   276
  end
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   277
    handle TERM _ => thm
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   278
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   279
fun abstract_domains_transfer thm =
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   280
  let
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   281
    fun dest prop =
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   282
      let
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   283
        val prems = Logic.strip_imp_prems prop
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   284
        val concl = HOLogic.dest_Trueprop (Logic.strip_imp_concl prop)
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   285
        val ((rel, x), y) = apfst Term.dest_comb (Term.dest_comb concl)
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   286
      in
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   287
        (x, fn x' =>
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   288
          Logic.list_implies (prems, HOLogic.mk_Trueprop (rel $ x' $ y)))
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   289
      end
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   290
  in
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   291
    gen_abstract_domains dest thm
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   292
  end
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   293
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   294
fun detect_transfer_rules thm =
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   295
  let
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   296
    fun is_transfer_rule tm = case (HOLogic.dest_Trueprop tm) of
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   297
      (Const (@{const_name HOL.eq}, _)) $ ((Const (@{const_name Domainp}, _)) $ _) $ _ => false
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   298
      | _ $ _ $ _ => true
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   299
      | _ => false
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   300
    fun safe_transfer_rule_conv ctm =
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   301
      if is_transfer_rule (term_of ctm) then safe_Rel_conv ctm else Conv.all_conv ctm
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   302
  in
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   303
    Conv.fconv_rule (Conv.prems_conv ~1 safe_transfer_rule_conv) thm
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   304
  end
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   305
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   306
(** Adding transfer domain rules **)
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   307
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   308
fun add_transfer_domain_thm thm = 
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   309
  (add_transfer_thm o abstract_equalities_domain o detect_transfer_rules) thm
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   310
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   311
fun del_transfer_domain_thm thm = 
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   312
  (del_transfer_thm o abstract_equalities_domain o detect_transfer_rules) thm
49975
faf4afed009f transfer package: more flexible handling of equality relations using is_equality predicate
huffman
parents: 49625
diff changeset
   313
faf4afed009f transfer package: more flexible handling of equality relations using is_equality predicate
huffman
parents: 49625
diff changeset
   314
(** Transfer proof method **)
47325
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
   315
47355
3d9d98e0f1a4 add bounded quantifier constant transfer_bforall, whose definition is unfolded after transfer
huffman
parents: 47327
diff changeset
   316
val post_simps =
47789
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   317
  @{thms transfer_forall_eq [symmetric]
47355
3d9d98e0f1a4 add bounded quantifier constant transfer_bforall, whose definition is unfolded after transfer
huffman
parents: 47327
diff changeset
   318
    transfer_implies_eq [symmetric] transfer_bforall_unfold}
3d9d98e0f1a4 add bounded quantifier constant transfer_bforall, whose definition is unfolded after transfer
huffman
parents: 47327
diff changeset
   319
47356
19fb95255ec9 transfer method generalizes over free variables in goal
huffman
parents: 47355
diff changeset
   320
fun gen_frees_tac keepers ctxt = SUBGOAL (fn (t, i) =>
19fb95255ec9 transfer method generalizes over free variables in goal
huffman
parents: 47355
diff changeset
   321
  let
48065
8aa05d38299a transfer method now avoids generalizing over free variables that are known to appear in registered transfer rules
huffman
parents: 48064
diff changeset
   322
    val keepers = keepers @ get_known_frees ctxt
47356
19fb95255ec9 transfer method generalizes over free variables in goal
huffman
parents: 47355
diff changeset
   323
    val vs = rev (Term.add_frees t [])
47568
98c8b7542b72 add option to transfer method for specifying variables not to generalize over
huffman
parents: 47523
diff changeset
   324
    val vs' = filter_out (member (op =) keepers) vs
47356
19fb95255ec9 transfer method generalizes over free variables in goal
huffman
parents: 47355
diff changeset
   325
  in
19fb95255ec9 transfer method generalizes over free variables in goal
huffman
parents: 47355
diff changeset
   326
    Induct.arbitrary_tac ctxt 0 vs' i
19fb95255ec9 transfer method generalizes over free variables in goal
huffman
parents: 47355
diff changeset
   327
  end)
19fb95255ec9 transfer method generalizes over free variables in goal
huffman
parents: 47355
diff changeset
   328
47789
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   329
fun mk_relT (T, U) = T --> U --> HOLogic.boolT
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   330
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   331
fun mk_Rel t =
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   332
  let val T = fastype_of t
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   333
  in Const (@{const_name Transfer.Rel}, T --> T) $ t end
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   334
52354
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   335
fun transfer_rule_of_terms (prj : typ * typ -> typ) ctxt tab t u =
47580
d99c883cdf2c use simpler method for preserving bound variable names in transfer tactic
huffman
parents: 47568
diff changeset
   336
  let
47789
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   337
    val thy = Proof_Context.theory_of ctxt
52354
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   338
    (* precondition: prj(T,U) must consist of only TFrees and type "fun" *)
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   339
    fun rel (T as Type ("fun", [T1, T2])) (U as Type ("fun", [U1, U2])) =
47789
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   340
        let
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   341
          val r1 = rel T1 U1
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   342
          val r2 = rel T2 U2
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   343
          val rT = fastype_of r1 --> fastype_of r2 --> mk_relT (T, U)
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   344
        in
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   345
          Const (@{const_name fun_rel}, rT) $ r1 $ r2
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   346
        end
52354
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   347
      | rel T U =
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   348
        let
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   349
          val (a, _) = dest_TFree (prj (T, U))
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   350
        in
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   351
          Free (the (AList.lookup (op =) tab a), mk_relT (T, U))
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   352
        end
47789
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   353
    fun zip _ thms (Bound i) (Bound _) = (nth thms i, [])
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   354
      | zip ctxt thms (Abs (x, T, t)) (Abs (y, U, u)) =
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   355
        let
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   356
          val ([x', y'], ctxt') = Variable.variant_fixes [x, y] ctxt
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   357
          val prop = mk_Rel (rel T U) $ Free (x', T) $ Free (y', U)
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   358
          val cprop = Thm.cterm_of thy (HOLogic.mk_Trueprop prop)
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   359
          val thm0 = Thm.assume cprop
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   360
          val (thm1, hyps) = zip ctxt' (thm0 :: thms) t u
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   361
          val ((r1, x), y) = apfst Thm.dest_comb (Thm.dest_comb (Thm.dest_arg cprop))
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   362
          val r2 = Thm.dest_fun2 (Thm.dest_arg (cprop_of thm1))
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   363
          val (a1, (b1, _)) = apsnd dest_funcT (dest_funcT (ctyp_of_term r1))
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   364
          val (a2, (b2, _)) = apsnd dest_funcT (dest_funcT (ctyp_of_term r2))
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   365
          val tinsts = [SOME a1, SOME b1, SOME a2, SOME b2]
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   366
          val insts = [SOME (Thm.dest_arg r1), SOME (Thm.dest_arg r2)]
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   367
          val rule = Drule.instantiate' tinsts insts @{thm Rel_abs}
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   368
          val thm2 = Thm.forall_intr x (Thm.forall_intr y (Thm.implies_intr cprop thm1))
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   369
        in
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   370
          (thm2 COMP rule, hyps)
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   371
        end
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   372
      | zip ctxt thms (f $ t) (g $ u) =
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   373
        let
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   374
          val (thm1, hyps1) = zip ctxt thms f g
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   375
          val (thm2, hyps2) = zip ctxt thms t u
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   376
        in
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   377
          (thm2 RS (thm1 RS @{thm Rel_app}), hyps1 @ hyps2)
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   378
        end
52354
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   379
      | zip _ _ t u =
47789
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   380
        let
52354
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   381
          val T = fastype_of t
47789
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   382
          val U = fastype_of u
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   383
          val prop = mk_Rel (rel T U) $ t $ u
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   384
          val cprop = Thm.cterm_of thy (HOLogic.mk_Trueprop prop)
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   385
        in
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   386
          (Thm.assume cprop, [cprop])
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   387
        end
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   388
    val r = mk_Rel (rel (fastype_of t) (fastype_of u))
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   389
    val goal = HOLogic.mk_Trueprop (r $ t $ u)
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   390
    val rename = Thm.trivial (cterm_of thy goal)
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   391
    val (thm, hyps) = zip ctxt [] t u
47580
d99c883cdf2c use simpler method for preserving bound variable names in transfer tactic
huffman
parents: 47568
diff changeset
   392
  in
47789
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   393
    Drule.implies_intr_list hyps (thm RS rename)
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   394
  end
47580
d99c883cdf2c use simpler method for preserving bound variable names in transfer tactic
huffman
parents: 47568
diff changeset
   395
52354
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   396
(* create a lambda term of the same shape as the given term *)
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   397
fun skeleton (is_atom : term -> bool) ctxt t =
47325
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
   398
  let
48066
c6783c9b87bf transfer method now handles transfer rules for compound terms, e.g. locale-defined constants with hidden parameters
huffman
parents: 48065
diff changeset
   399
    fun dummy ctxt =
c6783c9b87bf transfer method now handles transfer rules for compound terms, e.g. locale-defined constants with hidden parameters
huffman
parents: 48065
diff changeset
   400
      let
c6783c9b87bf transfer method now handles transfer rules for compound terms, e.g. locale-defined constants with hidden parameters
huffman
parents: 48065
diff changeset
   401
        val (c, ctxt) = yield_singleton Variable.variant_fixes "a" ctxt
c6783c9b87bf transfer method now handles transfer rules for compound terms, e.g. locale-defined constants with hidden parameters
huffman
parents: 48065
diff changeset
   402
      in
c6783c9b87bf transfer method now handles transfer rules for compound terms, e.g. locale-defined constants with hidden parameters
huffman
parents: 48065
diff changeset
   403
        (Free (c, dummyT), ctxt)
c6783c9b87bf transfer method now handles transfer rules for compound terms, e.g. locale-defined constants with hidden parameters
huffman
parents: 48065
diff changeset
   404
      end
52354
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   405
    fun go (Bound i) ctxt = (Bound i, ctxt)
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   406
      | go (Abs (x, _, t)) ctxt =
48066
c6783c9b87bf transfer method now handles transfer rules for compound terms, e.g. locale-defined constants with hidden parameters
huffman
parents: 48065
diff changeset
   407
        let
52354
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   408
          val (t', ctxt) = go t ctxt
48066
c6783c9b87bf transfer method now handles transfer rules for compound terms, e.g. locale-defined constants with hidden parameters
huffman
parents: 48065
diff changeset
   409
        in
c6783c9b87bf transfer method now handles transfer rules for compound terms, e.g. locale-defined constants with hidden parameters
huffman
parents: 48065
diff changeset
   410
          (Abs (x, dummyT, t'), ctxt)
c6783c9b87bf transfer method now handles transfer rules for compound terms, e.g. locale-defined constants with hidden parameters
huffman
parents: 48065
diff changeset
   411
        end
52354
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   412
      | go (tu as (t $ u)) ctxt =
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   413
        if is_atom tu andalso not (Term.is_open tu) then dummy ctxt else
48066
c6783c9b87bf transfer method now handles transfer rules for compound terms, e.g. locale-defined constants with hidden parameters
huffman
parents: 48065
diff changeset
   414
        let
52354
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   415
          val (t', ctxt) = go t ctxt
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   416
          val (u', ctxt) = go u ctxt
48066
c6783c9b87bf transfer method now handles transfer rules for compound terms, e.g. locale-defined constants with hidden parameters
huffman
parents: 48065
diff changeset
   417
        in
c6783c9b87bf transfer method now handles transfer rules for compound terms, e.g. locale-defined constants with hidden parameters
huffman
parents: 48065
diff changeset
   418
          (t' $ u', ctxt)
c6783c9b87bf transfer method now handles transfer rules for compound terms, e.g. locale-defined constants with hidden parameters
huffman
parents: 48065
diff changeset
   419
        end
52354
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   420
      | go _ ctxt = dummy ctxt
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   421
  in
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   422
    go t ctxt |> fst |> Syntax.check_term ctxt |>
47789
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   423
      map_types (map_type_tfree (fn (a, _) => TFree (a, HOLogic.typeS)))
52354
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   424
  end
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   425
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   426
(** Monotonicity analysis **)
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   427
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   428
(* TODO: Put extensible table in theory data *)
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   429
val monotab =
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   430
  Symtab.make
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   431
    [(@{const_name transfer_implies}, [~1, 1]),
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   432
     (@{const_name transfer_forall}, [1])(*,
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   433
     (@{const_name implies}, [~1, 1]),
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   434
     (@{const_name All}, [1])*)]
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   435
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   436
(*
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   437
Function bool_insts determines the set of boolean-relation variables
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   438
that can be instantiated to implies, rev_implies, or iff.
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   439
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   440
Invariants: bool_insts p (t, u) requires that
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   441
  u :: _ => _ => ... => bool, and
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   442
  t is a skeleton of u
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   443
*)
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   444
fun bool_insts p (t, u) =
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   445
  let
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   446
    fun strip2 (t1 $ t2, u1 $ u2, tus) =
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   447
        strip2 (t1, u1, (t2, u2) :: tus)
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   448
      | strip2 x = x
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   449
    fun or3 ((a, b, c), (x, y, z)) = (a orelse x, b orelse y, c orelse z)
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   450
    fun go Ts p (Abs (_, T, t), Abs (_, _, u)) tab = go (T :: Ts) p (t, u) tab
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   451
      | go Ts p (t, u) tab =
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   452
        let
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   453
          val (a, _) = dest_TFree (Term.body_type (Term.fastype_of1 (Ts, t)))
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   454
          val (_, tf, tus) = strip2 (t, u, [])
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   455
          val ps_opt = case tf of Const (c, _) => Symtab.lookup monotab c | _ => NONE
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   456
          val tab1 =
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   457
            case ps_opt of
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   458
              SOME ps =>
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   459
              let
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   460
                val ps' = map (fn x => p * x) (take (length tus) ps)
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   461
              in
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   462
                fold I (map2 (go Ts) ps' tus) tab
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   463
              end
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   464
            | NONE => tab
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   465
          val tab2 = Symtab.make [(a, (p >= 0, p <= 0, is_none ps_opt))]
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   466
        in
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   467
          Symtab.join (K or3) (tab1, tab2)
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   468
        end
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   469
    val tab = go [] p (t, u) Symtab.empty
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   470
    fun f (a, (true, false, false)) = SOME (a, @{const implies})
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   471
      | f (a, (false, true, false)) = SOME (a, @{const rev_implies})
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   472
      | f (a, (true, true, _))      = SOME (a, HOLogic.eq_const HOLogic.boolT)
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   473
      | f _                         = NONE
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   474
  in
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   475
    map_filter f (Symtab.dest tab)
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   476
  end
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   477
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   478
fun transfer_rule_of_term ctxt equiv t : thm =
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   479
  let
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   480
    val compound_rhs = get_compound_rhs ctxt
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   481
    val is_rhs = not o null o Net.unify_term compound_rhs
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   482
    val s = skeleton is_rhs ctxt t
47789
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   483
    val frees = map fst (Term.add_frees s [])
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   484
    val tfrees = map fst (Term.add_tfrees s [])
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   485
    fun prep a = "R" ^ Library.unprefix "'" a
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   486
    val (rnames, ctxt') = Variable.variant_fixes (map prep tfrees) ctxt
52354
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   487
    val tab = tfrees ~~ rnames
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   488
    fun prep a = the (AList.lookup (op =) tab a)
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   489
    val thm = transfer_rule_of_terms fst ctxt' tab s t
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   490
    val binsts = bool_insts (if equiv then 0 else 1) (s, t)
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   491
    val cbool = @{ctyp bool}
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   492
    val relT = @{typ "bool => bool => bool"}
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   493
    val idx = Thm.maxidx_of thm + 1
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   494
    val thy = Proof_Context.theory_of ctxt
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   495
    fun tinst (a, _) = (ctyp_of thy (TVar ((a, idx), HOLogic.typeS)), cbool)
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   496
    fun inst (a, t) = (cterm_of thy (Var (Name.clean_index (prep a, idx), relT)), cterm_of thy t)
47789
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   497
  in
52354
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   498
    thm
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   499
      |> Thm.generalize (tfrees, rnames @ frees) idx
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   500
      |> Thm.instantiate (map tinst binsts, map inst binsts)
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   501
  end
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   502
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   503
fun transfer_rule_of_lhs ctxt t : thm =
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   504
  let
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   505
    val compound_lhs = get_compound_lhs ctxt
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   506
    val is_lhs = not o null o Net.unify_term compound_lhs
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   507
    val s = skeleton is_lhs ctxt t
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   508
    val frees = map fst (Term.add_frees s [])
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   509
    val tfrees = map fst (Term.add_tfrees s [])
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   510
    fun prep a = "R" ^ Library.unprefix "'" a
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   511
    val (rnames, ctxt') = Variable.variant_fixes (map prep tfrees) ctxt
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   512
    val tab = tfrees ~~ rnames
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   513
    fun prep a = the (AList.lookup (op =) tab a)
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   514
    val thm = transfer_rule_of_terms snd ctxt' tab t s
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   515
    val binsts = bool_insts 1 (s, t)
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   516
    val cbool = @{ctyp bool}
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   517
    val relT = @{typ "bool => bool => bool"}
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   518
    val idx = Thm.maxidx_of thm + 1
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   519
    val thy = Proof_Context.theory_of ctxt
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   520
    fun tinst (a, _) = (ctyp_of thy (TVar ((a, idx), HOLogic.typeS)), cbool)
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   521
    fun inst (a, t) = (cterm_of thy (Var (Name.clean_index (prep a, idx), relT)), cterm_of thy t)
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   522
  in
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   523
    thm
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   524
      |> Thm.generalize (tfrees, rnames @ frees) idx
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   525
      |> Thm.instantiate (map tinst binsts, map inst binsts)
47789
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   526
  end
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   527
51437
8739f8abbecb fixing transfer tactic - unfold fully identity relation by using relator_eq
kuncar
parents: 51374
diff changeset
   528
fun eq_tac eq_rules = TRY o REPEAT_ALL_NEW (resolve_tac eq_rules) THEN_ALL_NEW rtac @{thm is_equality_eq}
8739f8abbecb fixing transfer tactic - unfold fully identity relation by using relator_eq
kuncar
parents: 51374
diff changeset
   529
47789
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   530
fun transfer_tac equiv ctxt i =
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   531
  let
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   532
    val pre_simps = @{thms transfer_forall_eq transfer_implies_eq}
52354
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   533
    val start_rule =
47789
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   534
      if equiv then @{thm transfer_start} else @{thm transfer_start'}
48064
7bd9e18ce058 unify theory-data structures for transfer package
huffman
parents: 47803
diff changeset
   535
    val rules = get_transfer_raw ctxt
51437
8739f8abbecb fixing transfer tactic - unfold fully identity relation by using relator_eq
kuncar
parents: 51374
diff changeset
   536
    val eq_rules = get_relator_eq_raw ctxt
47803
2e3821e13d67 allow transfer tactic to leave extra unsolved subgoals if transfer rules are missing
huffman
parents: 47789
diff changeset
   537
    (* allow unsolved subgoals only for standard transfer method, not for transfer' *)
2e3821e13d67 allow transfer tactic to leave extra unsolved subgoals if transfer rules are missing
huffman
parents: 47789
diff changeset
   538
    val end_tac = if equiv then K all_tac else K no_tac
49977
3259ea7a52af transfer package: error message if preprocessing goal to object-logic formula fails
huffman
parents: 49976
diff changeset
   539
    val err_msg = "Transfer failed to convert goal to an object-logic formula"
3259ea7a52af transfer package: error message if preprocessing goal to object-logic formula fails
huffman
parents: 49976
diff changeset
   540
    fun main_tac (t, i) =
3259ea7a52af transfer package: error message if preprocessing goal to object-logic formula fails
huffman
parents: 49976
diff changeset
   541
      rtac start_rule i THEN
52354
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   542
      (rtac (transfer_rule_of_term ctxt equiv (HOLogic.dest_Trueprop t))
49977
3259ea7a52af transfer package: error message if preprocessing goal to object-logic formula fails
huffman
parents: 49976
diff changeset
   543
        THEN_ALL_NEW
51437
8739f8abbecb fixing transfer tactic - unfold fully identity relation by using relator_eq
kuncar
parents: 51374
diff changeset
   544
          (SOLVED' (REPEAT_ALL_NEW (resolve_tac rules) THEN_ALL_NEW (DETERM o eq_tac eq_rules))
49977
3259ea7a52af transfer package: error message if preprocessing goal to object-logic formula fails
huffman
parents: 49976
diff changeset
   545
            ORELSE' end_tac)) (i + 1)
3259ea7a52af transfer package: error message if preprocessing goal to object-logic formula fails
huffman
parents: 49976
diff changeset
   546
        handle TERM (_, ts) => raise TERM (err_msg, ts)
47325
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
   547
  in
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
   548
    EVERY
47789
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   549
      [rewrite_goal_tac pre_simps i THEN
49977
3259ea7a52af transfer package: error message if preprocessing goal to object-logic formula fails
huffman
parents: 49976
diff changeset
   550
       SUBGOAL main_tac i,
47325
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
   551
       (* FIXME: rewrite_goal_tac does unwanted eta-contraction *)
47355
3d9d98e0f1a4 add bounded quantifier constant transfer_bforall, whose definition is unfolded after transfer
huffman
parents: 47327
diff changeset
   552
       rewrite_goal_tac post_simps i,
52354
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   553
       Goal.norm_hhf_tac i]
47789
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   554
  end
47325
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
   555
47789
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   556
fun transfer_prover_tac ctxt = SUBGOAL (fn (t, i) =>
47325
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
   557
  let
47789
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   558
    val rhs = (snd o Term.dest_comb o HOLogic.dest_Trueprop) t
52354
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   559
    val rule1 = transfer_rule_of_term ctxt false rhs
48064
7bd9e18ce058 unify theory-data structures for transfer package
huffman
parents: 47803
diff changeset
   560
    val rules = get_transfer_raw ctxt
51437
8739f8abbecb fixing transfer tactic - unfold fully identity relation by using relator_eq
kuncar
parents: 51374
diff changeset
   561
    val eq_rules = get_relator_eq_raw ctxt
47325
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
   562
  in
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
   563
    EVERY
47789
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   564
      [CONVERSION prep_conv i,
47635
ebb79474262c rename 'correspondence' method to 'transfer_prover'
huffman
parents: 47618
diff changeset
   565
       rtac @{thm transfer_prover_start} i,
47789
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   566
       (rtac rule1 THEN_ALL_NEW
51437
8739f8abbecb fixing transfer tactic - unfold fully identity relation by using relator_eq
kuncar
parents: 51374
diff changeset
   567
         (REPEAT_ALL_NEW (resolve_tac rules) THEN_ALL_NEW (DETERM o eq_tac eq_rules))) (i+1),
47618
1568dadd598a make correspondence tactic more robust by replacing lhs with schematic variable before applying intro rules
huffman
parents: 47580
diff changeset
   568
       rtac @{thm refl} i]
47789
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   569
  end)
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   570
52354
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   571
(** Transfer attribute **)
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   572
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   573
fun transferred ctxt extra_rules thm =
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   574
  let
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   575
    val start_rule = @{thm transfer_start}
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   576
    val start_rule' = @{thm transfer_start'}
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   577
    val rules = extra_rules @ get_transfer_raw ctxt
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   578
    val eq_rules = get_relator_eq_raw ctxt
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   579
    val err_msg = "Transfer failed to convert goal to an object-logic formula"
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   580
    val pre_simps = @{thms transfer_forall_eq transfer_implies_eq}
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   581
    val thm1 = Drule.forall_intr_vars thm
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   582
    val instT = rev (Term.add_tvars (Thm.full_prop_of thm1) [])
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   583
                |> map (fn v as ((a, _), S) => (v, TFree (a, S)))
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   584
    val thm2 = thm1
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   585
      |> Thm.certify_instantiate (instT, [])
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   586
      |> Raw_Simplifier.rewrite_rule pre_simps
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   587
    val ctxt' = Variable.declare_names (Thm.full_prop_of thm2) ctxt
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   588
    val t = HOLogic.dest_Trueprop (Thm.concl_of thm2)
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   589
    val rule = transfer_rule_of_lhs ctxt' t
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   590
    val tac =
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   591
      resolve_tac [thm2 RS start_rule', thm2 RS start_rule] 1 THEN
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   592
      (rtac rule
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   593
        THEN_ALL_NEW
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   594
          (SOLVED' (REPEAT_ALL_NEW (resolve_tac rules)
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   595
            THEN_ALL_NEW (DETERM o eq_tac eq_rules)))) 1
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   596
        handle TERM (_, ts) => raise TERM (err_msg, ts)
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   597
    val thm3 = Goal.prove_internal [] @{cpat "Trueprop ?P"} (K tac)
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   598
    val tnames = map (fst o dest_TFree o snd) instT
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   599
  in
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   600
    thm3
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   601
      |> Raw_Simplifier.rewrite_rule post_simps
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   602
      |> Raw_Simplifier.norm_hhf
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   603
      |> Drule.generalize (tnames, [])
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   604
      |> Drule.zero_var_indexes
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   605
  end
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   606
(*
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   607
    handle THM _ => thm
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   608
*)
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   609
52358
f4c4bcb0d564 implement 'untransferred' attribute, which is like 'transferred' but works in the opposite direction
huffman
parents: 52354
diff changeset
   610
fun untransferred ctxt extra_rules thm =
f4c4bcb0d564 implement 'untransferred' attribute, which is like 'transferred' but works in the opposite direction
huffman
parents: 52354
diff changeset
   611
  let
f4c4bcb0d564 implement 'untransferred' attribute, which is like 'transferred' but works in the opposite direction
huffman
parents: 52354
diff changeset
   612
    val start_rule = @{thm untransfer_start}
f4c4bcb0d564 implement 'untransferred' attribute, which is like 'transferred' but works in the opposite direction
huffman
parents: 52354
diff changeset
   613
    val rules = extra_rules @ get_transfer_raw ctxt
f4c4bcb0d564 implement 'untransferred' attribute, which is like 'transferred' but works in the opposite direction
huffman
parents: 52354
diff changeset
   614
    val eq_rules = get_relator_eq_raw ctxt
f4c4bcb0d564 implement 'untransferred' attribute, which is like 'transferred' but works in the opposite direction
huffman
parents: 52354
diff changeset
   615
    val err_msg = "Transfer failed to convert goal to an object-logic formula"
f4c4bcb0d564 implement 'untransferred' attribute, which is like 'transferred' but works in the opposite direction
huffman
parents: 52354
diff changeset
   616
    val pre_simps = @{thms transfer_forall_eq transfer_implies_eq}
f4c4bcb0d564 implement 'untransferred' attribute, which is like 'transferred' but works in the opposite direction
huffman
parents: 52354
diff changeset
   617
    val thm1 = Drule.forall_intr_vars thm
f4c4bcb0d564 implement 'untransferred' attribute, which is like 'transferred' but works in the opposite direction
huffman
parents: 52354
diff changeset
   618
    val instT = rev (Term.add_tvars (Thm.full_prop_of thm1) [])
f4c4bcb0d564 implement 'untransferred' attribute, which is like 'transferred' but works in the opposite direction
huffman
parents: 52354
diff changeset
   619
                |> map (fn v as ((a, _), S) => (v, TFree (a, S)))
f4c4bcb0d564 implement 'untransferred' attribute, which is like 'transferred' but works in the opposite direction
huffman
parents: 52354
diff changeset
   620
    val thm2 = thm1
f4c4bcb0d564 implement 'untransferred' attribute, which is like 'transferred' but works in the opposite direction
huffman
parents: 52354
diff changeset
   621
      |> Thm.certify_instantiate (instT, [])
f4c4bcb0d564 implement 'untransferred' attribute, which is like 'transferred' but works in the opposite direction
huffman
parents: 52354
diff changeset
   622
      |> Raw_Simplifier.rewrite_rule pre_simps
f4c4bcb0d564 implement 'untransferred' attribute, which is like 'transferred' but works in the opposite direction
huffman
parents: 52354
diff changeset
   623
    val ctxt' = Variable.declare_names (Thm.full_prop_of thm2) ctxt
f4c4bcb0d564 implement 'untransferred' attribute, which is like 'transferred' but works in the opposite direction
huffman
parents: 52354
diff changeset
   624
    val t = HOLogic.dest_Trueprop (Thm.concl_of thm2)
f4c4bcb0d564 implement 'untransferred' attribute, which is like 'transferred' but works in the opposite direction
huffman
parents: 52354
diff changeset
   625
    val rule = transfer_rule_of_term ctxt' true t
f4c4bcb0d564 implement 'untransferred' attribute, which is like 'transferred' but works in the opposite direction
huffman
parents: 52354
diff changeset
   626
    val tac =
f4c4bcb0d564 implement 'untransferred' attribute, which is like 'transferred' but works in the opposite direction
huffman
parents: 52354
diff changeset
   627
      rtac (thm2 RS start_rule) 1 THEN
f4c4bcb0d564 implement 'untransferred' attribute, which is like 'transferred' but works in the opposite direction
huffman
parents: 52354
diff changeset
   628
      (rtac rule
f4c4bcb0d564 implement 'untransferred' attribute, which is like 'transferred' but works in the opposite direction
huffman
parents: 52354
diff changeset
   629
        THEN_ALL_NEW
f4c4bcb0d564 implement 'untransferred' attribute, which is like 'transferred' but works in the opposite direction
huffman
parents: 52354
diff changeset
   630
          (SOLVED' (REPEAT_ALL_NEW (resolve_tac rules)
f4c4bcb0d564 implement 'untransferred' attribute, which is like 'transferred' but works in the opposite direction
huffman
parents: 52354
diff changeset
   631
            THEN_ALL_NEW (DETERM o eq_tac eq_rules)))) 1
f4c4bcb0d564 implement 'untransferred' attribute, which is like 'transferred' but works in the opposite direction
huffman
parents: 52354
diff changeset
   632
        handle TERM (_, ts) => raise TERM (err_msg, ts)
f4c4bcb0d564 implement 'untransferred' attribute, which is like 'transferred' but works in the opposite direction
huffman
parents: 52354
diff changeset
   633
    val thm3 = Goal.prove_internal [] @{cpat "Trueprop ?P"} (K tac)
f4c4bcb0d564 implement 'untransferred' attribute, which is like 'transferred' but works in the opposite direction
huffman
parents: 52354
diff changeset
   634
    val tnames = map (fst o dest_TFree o snd) instT
f4c4bcb0d564 implement 'untransferred' attribute, which is like 'transferred' but works in the opposite direction
huffman
parents: 52354
diff changeset
   635
  in
f4c4bcb0d564 implement 'untransferred' attribute, which is like 'transferred' but works in the opposite direction
huffman
parents: 52354
diff changeset
   636
    thm3
f4c4bcb0d564 implement 'untransferred' attribute, which is like 'transferred' but works in the opposite direction
huffman
parents: 52354
diff changeset
   637
      |> Raw_Simplifier.rewrite_rule post_simps
f4c4bcb0d564 implement 'untransferred' attribute, which is like 'transferred' but works in the opposite direction
huffman
parents: 52354
diff changeset
   638
      |> Raw_Simplifier.norm_hhf
f4c4bcb0d564 implement 'untransferred' attribute, which is like 'transferred' but works in the opposite direction
huffman
parents: 52354
diff changeset
   639
      |> Drule.generalize (tnames, [])
f4c4bcb0d564 implement 'untransferred' attribute, which is like 'transferred' but works in the opposite direction
huffman
parents: 52354
diff changeset
   640
      |> Drule.zero_var_indexes
f4c4bcb0d564 implement 'untransferred' attribute, which is like 'transferred' but works in the opposite direction
huffman
parents: 52354
diff changeset
   641
  end
f4c4bcb0d564 implement 'untransferred' attribute, which is like 'transferred' but works in the opposite direction
huffman
parents: 52354
diff changeset
   642
47789
71a526ee569a implement transfer tactic with more scalable forward proof methods
huffman
parents: 47658
diff changeset
   643
(** Methods and attributes **)
47325
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
   644
47568
98c8b7542b72 add option to transfer method for specifying variables not to generalize over
huffman
parents: 47523
diff changeset
   645
val free = Args.context -- Args.term >> (fn (_, Free v) => v | (ctxt, t) =>
98c8b7542b72 add option to transfer method for specifying variables not to generalize over
huffman
parents: 47523
diff changeset
   646
  error ("Bad free variable: " ^ Syntax.string_of_term ctxt t))
98c8b7542b72 add option to transfer method for specifying variables not to generalize over
huffman
parents: 47523
diff changeset
   647
98c8b7542b72 add option to transfer method for specifying variables not to generalize over
huffman
parents: 47523
diff changeset
   648
val fixing = Scan.optional (Scan.lift (Args.$$$ "fixing" -- Args.colon)
98c8b7542b72 add option to transfer method for specifying variables not to generalize over
huffman
parents: 47523
diff changeset
   649
  |-- Scan.repeat free) []
98c8b7542b72 add option to transfer method for specifying variables not to generalize over
huffman
parents: 47523
diff changeset
   650
47658
7631f6f7873d enable variant of transfer method that proves an implication instead of an equivalence
huffman
parents: 47635
diff changeset
   651
fun transfer_method equiv : (Proof.context -> Method.method) context_parser =
47568
98c8b7542b72 add option to transfer method for specifying variables not to generalize over
huffman
parents: 47523
diff changeset
   652
  fixing >> (fn vs => fn ctxt =>
47658
7631f6f7873d enable variant of transfer method that proves an implication instead of an equivalence
huffman
parents: 47635
diff changeset
   653
    SIMPLE_METHOD' (gen_frees_tac vs ctxt THEN' transfer_tac equiv ctxt))
47325
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
   654
47635
ebb79474262c rename 'correspondence' method to 'transfer_prover'
huffman
parents: 47618
diff changeset
   655
val transfer_prover_method : (Proof.context -> Method.method) context_parser =
ebb79474262c rename 'correspondence' method to 'transfer_prover'
huffman
parents: 47618
diff changeset
   656
  Scan.succeed (fn ctxt => SIMPLE_METHOD' (transfer_prover_tac ctxt))
47325
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
   657
47635
ebb79474262c rename 'correspondence' method to 'transfer_prover'
huffman
parents: 47618
diff changeset
   658
(* Attribute for transfer rules *)
47325
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
   659
51956
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   660
val prep_rule = abstract_domains_transfer o abstract_equalities_transfer o Conv.fconv_rule prep_conv
47325
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
   661
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
   662
val transfer_add =
48064
7bd9e18ce058 unify theory-data structures for transfer package
huffman
parents: 47803
diff changeset
   663
  Thm.declaration_attribute (add_transfer_thm o prep_rule)
47325
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
   664
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
   665
val transfer_del =
48064
7bd9e18ce058 unify theory-data structures for transfer package
huffman
parents: 47803
diff changeset
   666
  Thm.declaration_attribute (del_transfer_thm o prep_rule)
47325
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
   667
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
   668
val transfer_attribute =
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
   669
  Attrib.add_del transfer_add transfer_del
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
   670
51956
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   671
(* Attributes for transfer domain rules *)
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   672
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   673
val transfer_domain_add = Thm.declaration_attribute add_transfer_domain_thm
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   674
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   675
val transfer_domain_del = Thm.declaration_attribute del_transfer_domain_thm
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   676
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   677
val transfer_domain_attribute =
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   678
  Attrib.add_del transfer_domain_add transfer_domain_del
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   679
52354
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   680
(* Attributes for transferred rules *)
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   681
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   682
fun transferred_attribute thms = Thm.rule_attribute
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   683
  (fn context => transferred (Context.proof_of context) thms)
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   684
52358
f4c4bcb0d564 implement 'untransferred' attribute, which is like 'transferred' but works in the opposite direction
huffman
parents: 52354
diff changeset
   685
fun untransferred_attribute thms = Thm.rule_attribute
f4c4bcb0d564 implement 'untransferred' attribute, which is like 'transferred' but works in the opposite direction
huffman
parents: 52354
diff changeset
   686
  (fn context => untransferred (Context.proof_of context) thms)
f4c4bcb0d564 implement 'untransferred' attribute, which is like 'transferred' but works in the opposite direction
huffman
parents: 52354
diff changeset
   687
52354
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   688
val transferred_attribute_parser =
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   689
  Attrib.thms >> transferred_attribute
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   690
52358
f4c4bcb0d564 implement 'untransferred' attribute, which is like 'transferred' but works in the opposite direction
huffman
parents: 52354
diff changeset
   691
val untransferred_attribute_parser =
f4c4bcb0d564 implement 'untransferred' attribute, which is like 'transferred' but works in the opposite direction
huffman
parents: 52354
diff changeset
   692
  Attrib.thms >> untransferred_attribute
f4c4bcb0d564 implement 'untransferred' attribute, which is like 'transferred' but works in the opposite direction
huffman
parents: 52354
diff changeset
   693
47325
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
   694
(* Theory setup *)
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
   695
49975
faf4afed009f transfer package: more flexible handling of equality relations using is_equality predicate
huffman
parents: 49625
diff changeset
   696
val relator_eq_setup =
faf4afed009f transfer package: more flexible handling of equality relations using is_equality predicate
huffman
parents: 49625
diff changeset
   697
  let
faf4afed009f transfer package: more flexible handling of equality relations using is_equality predicate
huffman
parents: 49625
diff changeset
   698
    val name = @{binding relator_eq}
faf4afed009f transfer package: more flexible handling of equality relations using is_equality predicate
huffman
parents: 49625
diff changeset
   699
    fun add_thm thm = Data.map (map_relator_eq (Item_Net.update thm))
51437
8739f8abbecb fixing transfer tactic - unfold fully identity relation by using relator_eq
kuncar
parents: 51374
diff changeset
   700
      #> Data.map (map_relator_eq_raw (Item_Net.update (abstract_equalities_relator_eq thm)))
49975
faf4afed009f transfer package: more flexible handling of equality relations using is_equality predicate
huffman
parents: 49625
diff changeset
   701
    fun del_thm thm = Data.map (map_relator_eq (Item_Net.remove thm))
51437
8739f8abbecb fixing transfer tactic - unfold fully identity relation by using relator_eq
kuncar
parents: 51374
diff changeset
   702
      #> Data.map (map_relator_eq_raw (Item_Net.remove (abstract_equalities_relator_eq thm)))
49975
faf4afed009f transfer package: more flexible handling of equality relations using is_equality predicate
huffman
parents: 49625
diff changeset
   703
    val add = Thm.declaration_attribute add_thm
faf4afed009f transfer package: more flexible handling of equality relations using is_equality predicate
huffman
parents: 49625
diff changeset
   704
    val del = Thm.declaration_attribute del_thm
faf4afed009f transfer package: more flexible handling of equality relations using is_equality predicate
huffman
parents: 49625
diff changeset
   705
    val text = "declaration of relator equality rule (used by transfer method)"
faf4afed009f transfer package: more flexible handling of equality relations using is_equality predicate
huffman
parents: 49625
diff changeset
   706
    val content = Item_Net.content o #relator_eq o Data.get
faf4afed009f transfer package: more flexible handling of equality relations using is_equality predicate
huffman
parents: 49625
diff changeset
   707
  in
faf4afed009f transfer package: more flexible handling of equality relations using is_equality predicate
huffman
parents: 49625
diff changeset
   708
    Attrib.setup name (Attrib.add_del add del) text
faf4afed009f transfer package: more flexible handling of equality relations using is_equality predicate
huffman
parents: 49625
diff changeset
   709
    #> Global_Theory.add_thms_dynamic (name, content)
faf4afed009f transfer package: more flexible handling of equality relations using is_equality predicate
huffman
parents: 49625
diff changeset
   710
  end
faf4afed009f transfer package: more flexible handling of equality relations using is_equality predicate
huffman
parents: 49625
diff changeset
   711
51956
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   712
val relator_domain_setup =
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   713
  let
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   714
    val name = @{binding relator_domain}
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   715
    fun add_thm thm = Data.map (map_relator_domain (Item_Net.update thm))
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   716
      #> add_transfer_domain_thm thm
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   717
    fun del_thm thm = Data.map (map_relator_domain (Item_Net.remove thm))
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   718
      #> del_transfer_domain_thm thm
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   719
    val add = Thm.declaration_attribute add_thm
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   720
    val del = Thm.declaration_attribute del_thm
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   721
    val text = "declaration of relator domain rule (used by transfer method)"
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   722
    val content = Item_Net.content o #relator_domain o Data.get
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   723
  in
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   724
    Attrib.setup name (Attrib.add_del add del) text
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   725
    #> Global_Theory.add_thms_dynamic (name, content)
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   726
  end
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   727
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   728
47325
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
   729
val setup =
48064
7bd9e18ce058 unify theory-data structures for transfer package
huffman
parents: 47803
diff changeset
   730
  relator_eq_setup
51956
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   731
  #> relator_domain_setup
47325
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
   732
  #> Attrib.setup @{binding transfer_rule} transfer_attribute
47635
ebb79474262c rename 'correspondence' method to 'transfer_prover'
huffman
parents: 47618
diff changeset
   733
     "transfer rule for transfer method"
48064
7bd9e18ce058 unify theory-data structures for transfer package
huffman
parents: 47803
diff changeset
   734
  #> Global_Theory.add_thms_dynamic
7bd9e18ce058 unify theory-data structures for transfer package
huffman
parents: 47803
diff changeset
   735
     (@{binding transfer_raw}, Item_Net.content o #transfer_raw o Data.get)
51956
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   736
  #> Attrib.setup @{binding transfer_domain_rule} transfer_domain_attribute
a4d81cdebf8b better support for domains in Lifting/Transfer = replace Domainp T by the actual invariant in a transferred goal
kuncar
parents: 51955
diff changeset
   737
     "transfer domain rule for transfer method"
52354
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   738
  #> Attrib.setup @{binding transferred} transferred_attribute_parser
acb4f932dd24 implement 'transferred' attribute for transfer package, with support for monotonicity of !!/==>
huffman
parents: 51996
diff changeset
   739
     "raw theorem transferred to abstract theorem using transfer rules"
52358
f4c4bcb0d564 implement 'untransferred' attribute, which is like 'transferred' but works in the opposite direction
huffman
parents: 52354
diff changeset
   740
  #> Attrib.setup @{binding untransferred} untransferred_attribute_parser
f4c4bcb0d564 implement 'untransferred' attribute, which is like 'transferred' but works in the opposite direction
huffman
parents: 52354
diff changeset
   741
     "abstract theorem transferred to raw theorem using transfer rules"
51437
8739f8abbecb fixing transfer tactic - unfold fully identity relation by using relator_eq
kuncar
parents: 51374
diff changeset
   742
  #> Global_Theory.add_thms_dynamic
8739f8abbecb fixing transfer tactic - unfold fully identity relation by using relator_eq
kuncar
parents: 51374
diff changeset
   743
     (@{binding relator_eq_raw}, Item_Net.content o #relator_eq_raw o Data.get)
47658
7631f6f7873d enable variant of transfer method that proves an implication instead of an equivalence
huffman
parents: 47635
diff changeset
   744
  #> Method.setup @{binding transfer} (transfer_method true)
7631f6f7873d enable variant of transfer method that proves an implication instead of an equivalence
huffman
parents: 47635
diff changeset
   745
     "generic theorem transfer method"
7631f6f7873d enable variant of transfer method that proves an implication instead of an equivalence
huffman
parents: 47635
diff changeset
   746
  #> Method.setup @{binding transfer'} (transfer_method false)
47325
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
   747
     "generic theorem transfer method"
47635
ebb79474262c rename 'correspondence' method to 'transfer_prover'
huffman
parents: 47618
diff changeset
   748
  #> Method.setup @{binding transfer_prover} transfer_prover_method
ebb79474262c rename 'correspondence' method to 'transfer_prover'
huffman
parents: 47618
diff changeset
   749
     "for proving transfer rules"
47325
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
   750
ec6187036495 new transfer proof method
huffman
parents:
diff changeset
   751
end