src/ZF/ex/Comb.ML
author paulson
Fri, 03 Jan 1997 15:01:55 +0100
changeset 2469 b50b8c0eec01
parent 1732 38776e927da8
child 2496 40efb87985b5
permissions -rw-r--r--
Implicit simpsets and clasets for FOL and ZF
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
1461
6bcb44e4d6e5 expanded tabs
clasohm
parents: 782
diff changeset
     1
(*  Title:      ZF/ex/comb.ML
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
     2
    ID:         $Id$
1461
6bcb44e4d6e5 expanded tabs
clasohm
parents: 782
diff changeset
     3
    Author:     Lawrence C Paulson
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
     4
    Copyright   1993  University of Cambridge
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
     5
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
     6
Combinatory Logic example: the Church-Rosser Theorem
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
     7
Curiously, combinators do not include free variables.
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
     8
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
     9
Example taken from
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
    10
    J. Camilleri and T. F. Melham.
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
    11
    Reasoning with Inductively Defined Relations in the HOL Theorem Prover.
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
    12
    Report 265, University of Cambridge Computer Laboratory, 1992.
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
    13
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
    14
HOL system proofs may be found in
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
    15
/usr/groups/theory/hvg-aftp/contrib/rule-induction/cl.ml
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
    16
*)
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
    17
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
    18
open Comb;
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
    19
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
    20
val [_,_,comb_Ap] = comb.intrs;
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
    21
val Ap_E = comb.mk_cases comb.con_defs "p#q : comb";
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
    22
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
    23
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
    24
(*** Results about Contraction ***)
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
    25
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
    26
(*For type checking: replaces a-1->b by a,b:comb *)
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
    27
val contract_combE2 = contract.dom_subset RS subsetD RS SigmaE2;
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
    28
val contract_combD1 = contract.dom_subset RS subsetD RS SigmaD1;
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
    29
val contract_combD2 = contract.dom_subset RS subsetD RS SigmaD2;
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
    30
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
    31
goal Comb.thy "field(contract) = comb";
2469
b50b8c0eec01 Implicit simpsets and clasets for FOL and ZF
paulson
parents: 1732
diff changeset
    32
by (fast_tac (!claset addIs [equalityI,contract.K] addSEs [contract_combE2]) 1);
760
f0200e91b272 added qed and qed_goal[w]
clasohm
parents: 515
diff changeset
    33
qed "field_contract_eq";
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
    34
782
200a16083201 added bind_thm for theorems defined by "standard ..."
clasohm
parents: 760
diff changeset
    35
bind_thm ("reduction_refl",
200a16083201 added bind_thm for theorems defined by "standard ..."
clasohm
parents: 760
diff changeset
    36
    (field_contract_eq RS equalityD2 RS subsetD RS rtrancl_refl));
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
    37
782
200a16083201 added bind_thm for theorems defined by "standard ..."
clasohm
parents: 760
diff changeset
    38
bind_thm ("rtrancl_into_rtrancl2",
200a16083201 added bind_thm for theorems defined by "standard ..."
clasohm
parents: 760
diff changeset
    39
    (r_into_rtrancl RS (trans_rtrancl RS transD)));
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
    40
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
    41
val reduction_rls = [reduction_refl, contract.K, contract.S, 
1461
6bcb44e4d6e5 expanded tabs
clasohm
parents: 782
diff changeset
    42
                     contract.K RS rtrancl_into_rtrancl2,
6bcb44e4d6e5 expanded tabs
clasohm
parents: 782
diff changeset
    43
                     contract.S RS rtrancl_into_rtrancl2,
6bcb44e4d6e5 expanded tabs
clasohm
parents: 782
diff changeset
    44
                     contract.Ap1 RS rtrancl_into_rtrancl2,
6bcb44e4d6e5 expanded tabs
clasohm
parents: 782
diff changeset
    45
                     contract.Ap2 RS rtrancl_into_rtrancl2];
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
    46
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
    47
(*Example only: not used*)
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
    48
goalw Comb.thy [I_def] "!!p. p:comb ==> I#p ---> p";
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
    49
by (REPEAT (ares_tac (comb.intrs @ reduction_rls) 1));
782
200a16083201 added bind_thm for theorems defined by "standard ..."
clasohm
parents: 760
diff changeset
    50
qed "reduce_I";
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
    51
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
    52
goalw Comb.thy [I_def] "I: comb";
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
    53
by (REPEAT (ares_tac comb.intrs 1));
760
f0200e91b272 added qed and qed_goal[w]
clasohm
parents: 515
diff changeset
    54
qed "comb_I";
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
    55
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
    56
(** Non-contraction results **)
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
    57
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
    58
(*Derive a case for each combinator constructor*)
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
    59
val K_contractE = contract.mk_cases comb.con_defs "K -1-> r";
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
    60
val S_contractE = contract.mk_cases comb.con_defs "S -1-> r";
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
    61
val Ap_contractE = contract.mk_cases comb.con_defs "p#q -1-> r";
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
    62
2469
b50b8c0eec01 Implicit simpsets and clasets for FOL and ZF
paulson
parents: 1732
diff changeset
    63
AddSIs comb.intrs;
b50b8c0eec01 Implicit simpsets and clasets for FOL and ZF
paulson
parents: 1732
diff changeset
    64
AddIs  contract.intrs;
b50b8c0eec01 Implicit simpsets and clasets for FOL and ZF
paulson
parents: 1732
diff changeset
    65
AddSEs [contract_combD1,contract_combD2];     (*type checking*)
b50b8c0eec01 Implicit simpsets and clasets for FOL and ZF
paulson
parents: 1732
diff changeset
    66
AddSEs [K_contractE, S_contractE, Ap_contractE];
b50b8c0eec01 Implicit simpsets and clasets for FOL and ZF
paulson
parents: 1732
diff changeset
    67
AddSEs comb.free_SEs;
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
    68
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
    69
goalw Comb.thy [I_def] "!!r. I -1-> r ==> P";
2469
b50b8c0eec01 Implicit simpsets and clasets for FOL and ZF
paulson
parents: 1732
diff changeset
    70
by (Fast_tac 1);
782
200a16083201 added bind_thm for theorems defined by "standard ..."
clasohm
parents: 760
diff changeset
    71
qed "I_contract_E";
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
    72
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
    73
goal Comb.thy "!!p r. K#p -1-> r ==> (EX q. r = K#q & p -1-> q)";
2469
b50b8c0eec01 Implicit simpsets and clasets for FOL and ZF
paulson
parents: 1732
diff changeset
    74
by (Fast_tac 1);
782
200a16083201 added bind_thm for theorems defined by "standard ..."
clasohm
parents: 760
diff changeset
    75
qed "K1_contractD";
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
    76
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
    77
goal Comb.thy "!!p r. [| p ---> q;  r: comb |] ==> p#r ---> q#r";
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
    78
by (forward_tac [rtrancl_type RS subsetD RS SigmaD1] 1);
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
    79
by (dtac (field_contract_eq RS equalityD1 RS subsetD) 1);
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
    80
by (etac rtrancl_induct 1);
2469
b50b8c0eec01 Implicit simpsets and clasets for FOL and ZF
paulson
parents: 1732
diff changeset
    81
by (fast_tac (!claset addIs reduction_rls) 1);
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
    82
by (etac (trans_rtrancl RS transD) 1);
2469
b50b8c0eec01 Implicit simpsets and clasets for FOL and ZF
paulson
parents: 1732
diff changeset
    83
by (fast_tac (!claset addIs reduction_rls) 1);
782
200a16083201 added bind_thm for theorems defined by "standard ..."
clasohm
parents: 760
diff changeset
    84
qed "Ap_reduce1";
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
    85
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
    86
goal Comb.thy "!!p r. [| p ---> q;  r: comb |] ==> r#p ---> r#q";
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
    87
by (forward_tac [rtrancl_type RS subsetD RS SigmaD1] 1);
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
    88
by (dtac (field_contract_eq RS equalityD1 RS subsetD) 1);
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
    89
by (etac rtrancl_induct 1);
2469
b50b8c0eec01 Implicit simpsets and clasets for FOL and ZF
paulson
parents: 1732
diff changeset
    90
by (fast_tac (!claset addIs reduction_rls) 1);
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
    91
by (etac (trans_rtrancl RS transD) 1);
2469
b50b8c0eec01 Implicit simpsets and clasets for FOL and ZF
paulson
parents: 1732
diff changeset
    92
by (fast_tac (!claset addIs reduction_rls) 1);
782
200a16083201 added bind_thm for theorems defined by "standard ..."
clasohm
parents: 760
diff changeset
    93
qed "Ap_reduce2";
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
    94
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
    95
(** Counterexample to the diamond property for -1-> **)
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
    96
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
    97
goal Comb.thy "K#I#(I#I) -1-> I";
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
    98
by (REPEAT (ares_tac [contract.K, comb_I, comb_Ap] 1));
782
200a16083201 added bind_thm for theorems defined by "standard ..."
clasohm
parents: 760
diff changeset
    99
qed "KIII_contract1";
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   100
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   101
goalw Comb.thy [I_def] "K#I#(I#I) -1-> K#I#((K#I)#(K#I))";
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   102
by (DEPTH_SOLVE (resolve_tac (comb.intrs @ contract.intrs) 1));
782
200a16083201 added bind_thm for theorems defined by "standard ..."
clasohm
parents: 760
diff changeset
   103
qed "KIII_contract2";
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   104
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   105
goal Comb.thy "K#I#((K#I)#(K#I)) -1-> I";
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   106
by (REPEAT (ares_tac (comb.intrs @ [contract.K, comb_I]) 1));
782
200a16083201 added bind_thm for theorems defined by "standard ..."
clasohm
parents: 760
diff changeset
   107
qed "KIII_contract3";
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   108
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   109
goalw Comb.thy [diamond_def] "~ diamond(contract)";
2469
b50b8c0eec01 Implicit simpsets and clasets for FOL and ZF
paulson
parents: 1732
diff changeset
   110
by (fast_tac (!claset addIs [KIII_contract1,KIII_contract2,KIII_contract3]
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   111
                    addSEs [I_contract_E]) 1);
782
200a16083201 added bind_thm for theorems defined by "standard ..."
clasohm
parents: 760
diff changeset
   112
qed "not_diamond_contract";
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   113
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
   114
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
   115
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   116
(*** Results about Parallel Contraction ***)
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   117
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   118
(*For type checking: replaces a=1=>b by a,b:comb *)
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   119
val parcontract_combE2 = parcontract.dom_subset RS subsetD RS SigmaE2;
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   120
val parcontract_combD1 = parcontract.dom_subset RS subsetD RS SigmaD1;
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   121
val parcontract_combD2 = parcontract.dom_subset RS subsetD RS SigmaD2;
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   122
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   123
goal Comb.thy "field(parcontract) = comb";
2469
b50b8c0eec01 Implicit simpsets and clasets for FOL and ZF
paulson
parents: 1732
diff changeset
   124
by (fast_tac (!claset addIs [equalityI, parcontract.K] 
1461
6bcb44e4d6e5 expanded tabs
clasohm
parents: 782
diff changeset
   125
                    addSEs [parcontract_combE2]) 1);
782
200a16083201 added bind_thm for theorems defined by "standard ..."
clasohm
parents: 760
diff changeset
   126
qed "field_parcontract_eq";
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   127
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   128
(*Derive a case for each combinator constructor*)
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   129
val K_parcontractE = parcontract.mk_cases comb.con_defs "K =1=> r";
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   130
val S_parcontractE = parcontract.mk_cases comb.con_defs "S =1=> r";
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   131
val Ap_parcontractE = parcontract.mk_cases comb.con_defs "p#q =1=> r";
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   132
2469
b50b8c0eec01 Implicit simpsets and clasets for FOL and ZF
paulson
parents: 1732
diff changeset
   133
AddSIs comb.intrs;
b50b8c0eec01 Implicit simpsets and clasets for FOL and ZF
paulson
parents: 1732
diff changeset
   134
AddIs  parcontract.intrs;
b50b8c0eec01 Implicit simpsets and clasets for FOL and ZF
paulson
parents: 1732
diff changeset
   135
AddSEs [Ap_E, K_parcontractE, S_parcontractE, Ap_parcontractE];
b50b8c0eec01 Implicit simpsets and clasets for FOL and ZF
paulson
parents: 1732
diff changeset
   136
AddSEs [parcontract_combD1, parcontract_combD2];     (*type checking*)
b50b8c0eec01 Implicit simpsets and clasets for FOL and ZF
paulson
parents: 1732
diff changeset
   137
AddSEs comb.free_SEs;
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   138
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   139
(*** Basic properties of parallel contraction ***)
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   140
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   141
goal Comb.thy "!!p r. K#p =1=> r ==> (EX p'. r = K#p' & p =1=> p')";
2469
b50b8c0eec01 Implicit simpsets and clasets for FOL and ZF
paulson
parents: 1732
diff changeset
   142
by (Fast_tac 1);
782
200a16083201 added bind_thm for theorems defined by "standard ..."
clasohm
parents: 760
diff changeset
   143
qed "K1_parcontractD";
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   144
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   145
goal Comb.thy "!!p r. S#p =1=> r ==> (EX p'. r = S#p' & p =1=> p')";
2469
b50b8c0eec01 Implicit simpsets and clasets for FOL and ZF
paulson
parents: 1732
diff changeset
   146
by (Fast_tac 1);
782
200a16083201 added bind_thm for theorems defined by "standard ..."
clasohm
parents: 760
diff changeset
   147
qed "S1_parcontractD";
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   148
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   149
goal Comb.thy
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   150
 "!!p q r. S#p#q =1=> r ==> (EX p' q'. r = S#p'#q' & p =1=> p' & q =1=> q')";
2469
b50b8c0eec01 Implicit simpsets and clasets for FOL and ZF
paulson
parents: 1732
diff changeset
   151
by (fast_tac (!claset addSDs [S1_parcontractD]) 1);
782
200a16083201 added bind_thm for theorems defined by "standard ..."
clasohm
parents: 760
diff changeset
   152
qed "S2_parcontractD";
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   153
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   154
(*Church-Rosser property for parallel contraction*)
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   155
goalw Comb.thy [diamond_def] "diamond(parcontract)";
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   156
by (rtac (impI RS allI RS allI) 1);
1732
38776e927da8 Updated for new form of induction rules
paulson
parents: 1692
diff changeset
   157
by (etac parcontract.induct 1);
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   158
by (ALLGOALS 
2469
b50b8c0eec01 Implicit simpsets and clasets for FOL and ZF
paulson
parents: 1732
diff changeset
   159
    (fast_tac (!claset addSDs [K1_parcontractD,S2_parcontractD])));
782
200a16083201 added bind_thm for theorems defined by "standard ..."
clasohm
parents: 760
diff changeset
   160
qed "diamond_parcontract";
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   161
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   162
(*** Transitive closure preserves the Church-Rosser property ***)
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
   163
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   164
goalw Comb.thy [diamond_def]
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   165
    "!!x y r. [| diamond(r);  <x,y>:r^+ |] ==> \
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   166
\    ALL y'. <x,y'>:r --> (EX z. <y',z>: r^+ & <y,z>: r)";
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   167
by (etac trancl_induct 1);
2469
b50b8c0eec01 Implicit simpsets and clasets for FOL and ZF
paulson
parents: 1732
diff changeset
   168
by (fast_tac (!claset addIs [r_into_trancl]) 1);
b50b8c0eec01 Implicit simpsets and clasets for FOL and ZF
paulson
parents: 1732
diff changeset
   169
by (slow_best_tac (!claset addSDs [spec RS mp]
1461
6bcb44e4d6e5 expanded tabs
clasohm
parents: 782
diff changeset
   170
                         addIs  [r_into_trancl, trans_trancl RS transD]) 1);
1692
5324be24a5fa Renaming of a lemma
paulson
parents: 1461
diff changeset
   171
val diamond_strip_lemmaE = result() RS spec RS mp RS exE;
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   172
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   173
val [major] = goal Comb.thy "diamond(r) ==> diamond(r^+)";
1461
6bcb44e4d6e5 expanded tabs
clasohm
parents: 782
diff changeset
   174
by (rewtac diamond_def);  (*unfold only in goal, not in premise!*)
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   175
by (rtac (impI RS allI RS allI) 1);
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   176
by (etac trancl_induct 1);
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   177
by (ALLGOALS
2469
b50b8c0eec01 Implicit simpsets and clasets for FOL and ZF
paulson
parents: 1732
diff changeset
   178
    (slow_best_tac (!claset addIs [r_into_trancl, trans_trancl RS transD]
1692
5324be24a5fa Renaming of a lemma
paulson
parents: 1461
diff changeset
   179
                          addEs [major RS diamond_strip_lemmaE])));
782
200a16083201 added bind_thm for theorems defined by "standard ..."
clasohm
parents: 760
diff changeset
   180
qed "diamond_trancl";
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   181
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   182
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   183
(*** Equivalence of p--->q and p===>q ***)
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   184
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   185
goal Comb.thy "!!p q. p-1->q ==> p=1=>q";
1732
38776e927da8 Updated for new form of induction rules
paulson
parents: 1692
diff changeset
   186
by (etac contract.induct 1);
2469
b50b8c0eec01 Implicit simpsets and clasets for FOL and ZF
paulson
parents: 1732
diff changeset
   187
by (ALLGOALS (fast_tac (!claset)));
782
200a16083201 added bind_thm for theorems defined by "standard ..."
clasohm
parents: 760
diff changeset
   188
qed "contract_imp_parcontract";
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
   189
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   190
goal Comb.thy "!!p q. p--->q ==> p===>q";
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   191
by (forward_tac [rtrancl_type RS subsetD RS SigmaD1] 1);
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   192
by (dtac (field_contract_eq RS equalityD1 RS subsetD) 1);
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   193
by (etac rtrancl_induct 1);
2469
b50b8c0eec01 Implicit simpsets and clasets for FOL and ZF
paulson
parents: 1732
diff changeset
   194
by (fast_tac (!claset addIs [r_into_trancl]) 1);
b50b8c0eec01 Implicit simpsets and clasets for FOL and ZF
paulson
parents: 1732
diff changeset
   195
by (fast_tac (!claset addIs [contract_imp_parcontract, 
1461
6bcb44e4d6e5 expanded tabs
clasohm
parents: 782
diff changeset
   196
                           r_into_trancl, trans_trancl RS transD]) 1);
782
200a16083201 added bind_thm for theorems defined by "standard ..."
clasohm
parents: 760
diff changeset
   197
qed "reduce_imp_parreduce";
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   198
0
a5a9c433f639 Initial revision
clasohm
parents:
diff changeset
   199
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   200
goal Comb.thy "!!p q. p=1=>q ==> p--->q";
1732
38776e927da8 Updated for new form of induction rules
paulson
parents: 1692
diff changeset
   201
by (etac parcontract.induct 1);
2469
b50b8c0eec01 Implicit simpsets and clasets for FOL and ZF
paulson
parents: 1732
diff changeset
   202
by (fast_tac (!claset addIs reduction_rls) 1);
b50b8c0eec01 Implicit simpsets and clasets for FOL and ZF
paulson
parents: 1732
diff changeset
   203
by (fast_tac (!claset addIs reduction_rls) 1);
b50b8c0eec01 Implicit simpsets and clasets for FOL and ZF
paulson
parents: 1732
diff changeset
   204
by (fast_tac (!claset addIs reduction_rls) 1);
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   205
by (rtac (trans_rtrancl RS transD) 1);
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   206
by (ALLGOALS 
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   207
    (fast_tac 
2469
b50b8c0eec01 Implicit simpsets and clasets for FOL and ZF
paulson
parents: 1732
diff changeset
   208
     (!claset addIs [Ap_reduce1, Ap_reduce2]
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   209
                  addSEs [parcontract_combD1,parcontract_combD2])));
760
f0200e91b272 added qed and qed_goal[w]
clasohm
parents: 515
diff changeset
   210
qed "parcontract_imp_reduce";
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   211
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   212
goal Comb.thy "!!p q. p===>q ==> p--->q";
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   213
by (forward_tac [trancl_type RS subsetD RS SigmaD1] 1);
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   214
by (dtac (field_parcontract_eq RS equalityD1 RS subsetD) 1);
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   215
by (etac trancl_induct 1);
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   216
by (etac parcontract_imp_reduce 1);
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   217
by (etac (trans_rtrancl RS transD) 1);
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   218
by (etac parcontract_imp_reduce 1);
782
200a16083201 added bind_thm for theorems defined by "standard ..."
clasohm
parents: 760
diff changeset
   219
qed "parreduce_imp_reduce";
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   220
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   221
goal Comb.thy "p===>q <-> p--->q";
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   222
by (REPEAT (ares_tac [iffI, parreduce_imp_reduce, reduce_imp_parreduce] 1));
782
200a16083201 added bind_thm for theorems defined by "standard ..."
clasohm
parents: 760
diff changeset
   223
qed "parreduce_iff_reduce";
515
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   224
abcc438e7c27 installation of new inductive/datatype sections
lcp
parents: 486
diff changeset
   225
writeln"Reached end of file.";