src/HOL/ex/MT.ML
author berghofe
Tue, 25 Jun 1996 13:11:29 +0200
changeset 1824 44254696843a
parent 1820 e381e1c51689
child 2935 998cb95fdd43
permissions -rw-r--r--
Changed argument order of nat_rec.
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
1465
5d7a7e439cec expanded tabs
clasohm
parents: 1266
diff changeset
     1
(*  Title:      HOL/ex/MT.ML
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
     2
    ID:         $Id$
1465
5d7a7e439cec expanded tabs
clasohm
parents: 1266
diff changeset
     3
    Author:     Jacob Frost, Cambridge University Computer Laboratory
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
     4
    Copyright   1993  University of Cambridge
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
     5
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
     6
Based upon the article
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
     7
    Robin Milner and Mads Tofte,
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
     8
    Co-induction in Relational Semantics,
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
     9
    Theoretical Computer Science 87 (1991), pages 209-220.
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
    10
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
    11
Written up as
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
    12
    Jacob Frost, A Case Study of Co-induction in Isabelle/HOL
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
    13
    Report 308, Computer Lab, University of Cambridge (1993).
1047
5133479a37cf Simplified some proofs and made them work for new hyp_subst_tac.
lcp
parents: 972
diff changeset
    14
5133479a37cf Simplified some proofs and made them work for new hyp_subst_tac.
lcp
parents: 972
diff changeset
    15
NEEDS TO USE INDUCTIVE DEFS PACKAGE
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
    16
*)
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
    17
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
    18
open MT;
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
    19
1584
3d59c407bd36 Sets a lower value of Unify.search_bound
paulson
parents: 1465
diff changeset
    20
(*Limit cyclic unifications during monotonicity proofs*)
3d59c407bd36 Sets a lower value of Unify.search_bound
paulson
parents: 1465
diff changeset
    21
val orig_search_bound = !Unify.search_bound;
3d59c407bd36 Sets a lower value of Unify.search_bound
paulson
parents: 1465
diff changeset
    22
Unify.search_bound := 8;
3d59c407bd36 Sets a lower value of Unify.search_bound
paulson
parents: 1465
diff changeset
    23
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
    24
val prems = goal MT.thy "~a:{b} ==> ~a=b";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
    25
by (cut_facts_tac prems 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
    26
by (rtac notI 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
    27
by (dtac notE 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
    28
by (hyp_subst_tac 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
    29
by (rtac singletonI 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
    30
by (assume_tac 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
    31
qed "notsingletonI";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
    32
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
    33
(* ############################################################ *)
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
    34
(* Inference systems                                            *)
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
    35
(* ############################################################ *)
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
    36
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
    37
val infsys_mono_tac =
1820
e381e1c51689 Classical tactics now use default claset.
berghofe
parents: 1584
diff changeset
    38
  (rewtac subset_def) THEN (safe_tac (claset_of "HOL")) THEN (rtac ballI 1) THEN
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
    39
  (rtac CollectI 1) THEN (dtac CollectD 1) THEN
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
    40
  REPEAT 
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
    41
    ( (TRY ((etac disjE 1) THEN (rtac disjI2 2) THEN (rtac disjI1 1))) THEN
1820
e381e1c51689 Classical tactics now use default claset.
berghofe
parents: 1584
diff changeset
    42
      (REPEAT (etac exE 1)) THEN (REPEAT (rtac exI 1)) THEN (fast_tac ((claset_of "Fun")delrules [equalityI]) 1)
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
    43
    );
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
    44
972
e61b058d58d2 changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents: 969
diff changeset
    45
val prems = goal MT.thy "P a b ==> P (fst (a,b)) (snd (a,b))";
1266
3ae9fe3c0f68 added local simpsets
clasohm
parents: 1047
diff changeset
    46
by (simp_tac (!simpset addsimps prems) 1);
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
    47
qed "infsys_p1";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
    48
1047
5133479a37cf Simplified some proofs and made them work for new hyp_subst_tac.
lcp
parents: 972
diff changeset
    49
val prems = goal MT.thy "!!a b. P (fst (a,b)) (snd (a,b)) ==> P a b";
1266
3ae9fe3c0f68 added local simpsets
clasohm
parents: 1047
diff changeset
    50
by (Asm_full_simp_tac 1);
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
    51
qed "infsys_p2";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
    52
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
    53
val prems = goal MT.thy 
1047
5133479a37cf Simplified some proofs and made them work for new hyp_subst_tac.
lcp
parents: 972
diff changeset
    54
 "!!a. P a b c ==> P (fst(fst((a,b),c))) (snd(fst ((a,b),c))) (snd ((a,b),c))";
1266
3ae9fe3c0f68 added local simpsets
clasohm
parents: 1047
diff changeset
    55
by (Asm_full_simp_tac 1);
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
    56
qed "infsys_pp1";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
    57
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
    58
val prems = goal MT.thy 
1047
5133479a37cf Simplified some proofs and made them work for new hyp_subst_tac.
lcp
parents: 972
diff changeset
    59
 "!!a. P (fst(fst((a,b),c))) (snd(fst((a,b),c))) (snd((a,b),c)) ==> P a b c";
1266
3ae9fe3c0f68 added local simpsets
clasohm
parents: 1047
diff changeset
    60
by (Asm_full_simp_tac 1);
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
    61
qed "infsys_pp2";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
    62
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
    63
(* ############################################################ *)
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
    64
(* Fixpoints                                                    *)
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
    65
(* ############################################################ *)
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
    66
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
    67
(* Least fixpoints *)
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
    68
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
    69
val prems = goal MT.thy "[| mono(f); x:f(lfp(f)) |] ==> x:lfp(f)";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
    70
by (rtac subsetD 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
    71
by (rtac lfp_lemma2 1);
1047
5133479a37cf Simplified some proofs and made them work for new hyp_subst_tac.
lcp
parents: 972
diff changeset
    72
by (resolve_tac prems 1);
5133479a37cf Simplified some proofs and made them work for new hyp_subst_tac.
lcp
parents: 972
diff changeset
    73
by (resolve_tac prems 1);
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
    74
qed "lfp_intro2";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
    75
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
    76
val prems = goal MT.thy
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
    77
  " [| x:lfp(f); mono(f); !!y. y:f(lfp(f)) ==> P(y) |] ==> \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
    78
\   P(x)";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
    79
by (cut_facts_tac prems 1);
1047
5133479a37cf Simplified some proofs and made them work for new hyp_subst_tac.
lcp
parents: 972
diff changeset
    80
by (resolve_tac prems 1);
5133479a37cf Simplified some proofs and made them work for new hyp_subst_tac.
lcp
parents: 972
diff changeset
    81
by (rtac subsetD 1);
5133479a37cf Simplified some proofs and made them work for new hyp_subst_tac.
lcp
parents: 972
diff changeset
    82
by (rtac lfp_lemma3 1);
5133479a37cf Simplified some proofs and made them work for new hyp_subst_tac.
lcp
parents: 972
diff changeset
    83
by (assume_tac 1);
5133479a37cf Simplified some proofs and made them work for new hyp_subst_tac.
lcp
parents: 972
diff changeset
    84
by (assume_tac 1);
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
    85
qed "lfp_elim2";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
    86
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
    87
val prems = goal MT.thy
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
    88
  " [| x:lfp(f); mono(f); !!y. y:f(lfp(f) Int {x.P(x)}) ==> P(y) |] ==> \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
    89
\   P(x)";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
    90
by (cut_facts_tac prems 1);
1047
5133479a37cf Simplified some proofs and made them work for new hyp_subst_tac.
lcp
parents: 972
diff changeset
    91
by (etac induct 1);
5133479a37cf Simplified some proofs and made them work for new hyp_subst_tac.
lcp
parents: 972
diff changeset
    92
by (assume_tac 1);
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
    93
by (eresolve_tac prems 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
    94
qed "lfp_ind2";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
    95
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
    96
(* Greatest fixpoints *)
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
    97
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
    98
(* Note : "[| x:S; S <= f(S Un gfp(f)); mono(f) |] ==> x:gfp(f)" *)
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
    99
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   100
val [cih,monoh] = goal MT.thy "[| x:f({x} Un gfp(f)); mono(f) |] ==> x:gfp(f)";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   101
by (rtac (cih RSN (2,gfp_upperbound RS subsetD)) 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   102
by (rtac (monoh RS monoD) 1);
1047
5133479a37cf Simplified some proofs and made them work for new hyp_subst_tac.
lcp
parents: 972
diff changeset
   103
by (rtac (UnE RS subsetI) 1);
5133479a37cf Simplified some proofs and made them work for new hyp_subst_tac.
lcp
parents: 972
diff changeset
   104
by (assume_tac 1);
1820
e381e1c51689 Classical tactics now use default claset.
berghofe
parents: 1584
diff changeset
   105
by (fast_tac (!claset addSIs [cih]) 1);
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   106
by (rtac (monoh RS monoD RS subsetD) 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   107
by (rtac Un_upper2 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   108
by (etac (monoh RS gfp_lemma2 RS subsetD) 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   109
qed "gfp_coind2";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   110
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   111
val [gfph,monoh,caseh] = goal MT.thy 
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   112
  "[| x:gfp(f); mono(f); !! y. y:f(gfp(f)) ==> P(y) |] ==> P(x)";
1047
5133479a37cf Simplified some proofs and made them work for new hyp_subst_tac.
lcp
parents: 972
diff changeset
   113
by (rtac caseh 1);
5133479a37cf Simplified some proofs and made them work for new hyp_subst_tac.
lcp
parents: 972
diff changeset
   114
by (rtac subsetD 1);
5133479a37cf Simplified some proofs and made them work for new hyp_subst_tac.
lcp
parents: 972
diff changeset
   115
by (rtac gfp_lemma2 1);
5133479a37cf Simplified some proofs and made them work for new hyp_subst_tac.
lcp
parents: 972
diff changeset
   116
by (rtac monoh 1);
5133479a37cf Simplified some proofs and made them work for new hyp_subst_tac.
lcp
parents: 972
diff changeset
   117
by (rtac gfph 1);
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   118
qed "gfp_elim2";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   119
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   120
(* ############################################################ *)
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   121
(* Expressions                                                  *)
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   122
(* ############################################################ *)
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   123
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   124
val e_injs = [e_const_inj, e_var_inj, e_fn_inj, e_fix_inj, e_app_inj];
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   125
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   126
val e_disjs = 
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   127
  [ e_disj_const_var, 
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   128
    e_disj_const_fn, 
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   129
    e_disj_const_fix, 
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   130
    e_disj_const_app,
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   131
    e_disj_var_fn, 
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   132
    e_disj_var_fix, 
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   133
    e_disj_var_app, 
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   134
    e_disj_fn_fix, 
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   135
    e_disj_fn_app, 
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   136
    e_disj_fix_app
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   137
  ];
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   138
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   139
val e_disj_si = e_disjs @ (e_disjs RL [not_sym]);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   140
val e_disj_se = (e_disj_si RL [notE]);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   141
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   142
fun e_ext_cs cs = cs addSIs e_disj_si addSEs e_disj_se addSDs e_injs;
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   143
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   144
(* ############################################################ *)
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   145
(* Values                                                      *)
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   146
(* ############################################################ *)
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   147
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   148
val v_disjs = [v_disj_const_clos];
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   149
val v_disj_si = v_disjs @ (v_disjs RL [not_sym]);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   150
val v_disj_se = (v_disj_si RL [notE]);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   151
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   152
val v_injs = [v_const_inj, v_clos_inj];
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   153
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   154
fun v_ext_cs cs  = cs addSIs v_disj_si addSEs v_disj_se addSDs v_injs;
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   155
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   156
(* ############################################################ *)
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   157
(* Evaluations                                                  *)
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   158
(* ############################################################ *)
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   159
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   160
(* Monotonicity of eval_fun *)
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   161
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   162
goalw MT.thy [mono_def, eval_fun_def] "mono(eval_fun)";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   163
by infsys_mono_tac;
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   164
qed "eval_fun_mono";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   165
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   166
(* Introduction rules *)
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   167
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   168
goalw MT.thy [eval_def, eval_rel_def] "ve |- e_const(c) ---> v_const(c)";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   169
by (rtac lfp_intro2 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   170
by (rtac eval_fun_mono 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   171
by (rewtac eval_fun_def);
1820
e381e1c51689 Classical tactics now use default claset.
berghofe
parents: 1584
diff changeset
   172
by (Fast_tac 1);
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   173
qed "eval_const";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   174
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   175
val prems = goalw MT.thy [eval_def, eval_rel_def] 
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   176
  "ev:ve_dom(ve) ==> ve |- e_var(ev) ---> ve_app ve ev";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   177
by (cut_facts_tac prems 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   178
by (rtac lfp_intro2 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   179
by (rtac eval_fun_mono 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   180
by (rewtac eval_fun_def);
1820
e381e1c51689 Classical tactics now use default claset.
berghofe
parents: 1584
diff changeset
   181
by (Fast_tac 1);
1266
3ae9fe3c0f68 added local simpsets
clasohm
parents: 1047
diff changeset
   182
qed "eval_var2";
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   183
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   184
val prems = goalw MT.thy [eval_def, eval_rel_def] 
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   185
  "ve |- fn ev => e ---> v_clos(<|ev,e,ve|>)";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   186
by (cut_facts_tac prems 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   187
by (rtac lfp_intro2 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   188
by (rtac eval_fun_mono 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   189
by (rewtac eval_fun_def);
1820
e381e1c51689 Classical tactics now use default claset.
berghofe
parents: 1584
diff changeset
   190
by (Fast_tac 1);
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   191
qed "eval_fn";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   192
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   193
val prems = goalw MT.thy [eval_def, eval_rel_def] 
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   194
  " cl = <| ev1, e, ve + {ev2 |-> v_clos(cl)} |> ==> \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   195
\   ve |- fix ev2(ev1) = e ---> v_clos(cl)";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   196
by (cut_facts_tac prems 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   197
by (rtac lfp_intro2 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   198
by (rtac eval_fun_mono 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   199
by (rewtac eval_fun_def);
1820
e381e1c51689 Classical tactics now use default claset.
berghofe
parents: 1584
diff changeset
   200
by (Fast_tac 1);
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   201
qed "eval_fix";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   202
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   203
val prems = goalw MT.thy [eval_def, eval_rel_def]
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   204
  " [| ve |- e1 ---> v_const(c1); ve |- e2 ---> v_const(c2) |] ==> \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   205
\   ve |- e1 @ e2 ---> v_const(c_app c1 c2)";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   206
by (cut_facts_tac prems 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   207
by (rtac lfp_intro2 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   208
by (rtac eval_fun_mono 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   209
by (rewtac eval_fun_def);
1820
e381e1c51689 Classical tactics now use default claset.
berghofe
parents: 1584
diff changeset
   210
by (Fast_tac 1);
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   211
qed "eval_app1";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   212
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   213
val prems = goalw MT.thy [eval_def, eval_rel_def] 
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   214
  " [|  ve |- e1 ---> v_clos(<|xm,em,vem|>); \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   215
\       ve |- e2 ---> v2; \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   216
\       vem + {xm |-> v2} |- em ---> v \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   217
\   |] ==> \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   218
\   ve |- e1 @ e2 ---> v";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   219
by (cut_facts_tac prems 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   220
by (rtac lfp_intro2 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   221
by (rtac eval_fun_mono 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   222
by (rewtac eval_fun_def);
1820
e381e1c51689 Classical tactics now use default claset.
berghofe
parents: 1584
diff changeset
   223
by (fast_tac (!claset addSIs [disjI2]) 1);
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   224
qed "eval_app2";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   225
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   226
(* Strong elimination, induction on evaluations *)
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   227
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   228
val prems = goalw MT.thy [eval_def, eval_rel_def]
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   229
  " [| ve |- e ---> v; \
972
e61b058d58d2 changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents: 969
diff changeset
   230
\      !!ve c. P(((ve,e_const(c)),v_const(c))); \
e61b058d58d2 changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents: 969
diff changeset
   231
\      !!ev ve. ev:ve_dom(ve) ==> P(((ve,e_var(ev)),ve_app ve ev)); \
e61b058d58d2 changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents: 969
diff changeset
   232
\      !!ev ve e. P(((ve,fn ev => e),v_clos(<|ev,e,ve|>))); \
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   233
\      !!ev1 ev2 ve cl e. \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   234
\        cl = <| ev1, e, ve + {ev2 |-> v_clos(cl)} |> ==> \
972
e61b058d58d2 changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents: 969
diff changeset
   235
\        P(((ve,fix ev2(ev1) = e),v_clos(cl))); \
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   236
\      !!ve c1 c2 e1 e2. \
972
e61b058d58d2 changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents: 969
diff changeset
   237
\        [| P(((ve,e1),v_const(c1))); P(((ve,e2),v_const(c2))) |] ==> \
e61b058d58d2 changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents: 969
diff changeset
   238
\        P(((ve,e1 @ e2),v_const(c_app c1 c2))); \
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   239
\      !!ve vem xm e1 e2 em v v2. \
972
e61b058d58d2 changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents: 969
diff changeset
   240
\        [|  P(((ve,e1),v_clos(<|xm,em,vem|>))); \
e61b058d58d2 changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents: 969
diff changeset
   241
\            P(((ve,e2),v2)); \
e61b058d58d2 changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents: 969
diff changeset
   242
\            P(((vem + {xm |-> v2},em),v)) \
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   243
\        |] ==> \
972
e61b058d58d2 changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents: 969
diff changeset
   244
\        P(((ve,e1 @ e2),v)) \
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   245
\   |] ==> \
972
e61b058d58d2 changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents: 969
diff changeset
   246
\   P(((ve,e),v))";
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   247
by (resolve_tac (prems RL [lfp_ind2]) 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   248
by (rtac eval_fun_mono 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   249
by (rewtac eval_fun_def);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   250
by (dtac CollectD 1);
1820
e381e1c51689 Classical tactics now use default claset.
berghofe
parents: 1584
diff changeset
   251
by (safe_tac (!claset));
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   252
by (ALLGOALS (resolve_tac prems));
1820
e381e1c51689 Classical tactics now use default claset.
berghofe
parents: 1584
diff changeset
   253
by (ALLGOALS (Fast_tac));
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   254
qed "eval_ind0";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   255
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   256
val prems = goal MT.thy 
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   257
  " [| ve |- e ---> v; \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   258
\      !!ve c. P ve (e_const c) (v_const c); \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   259
\      !!ev ve. ev:ve_dom(ve) ==> P ve (e_var ev) (ve_app ve ev); \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   260
\      !!ev ve e. P ve (fn ev => e) (v_clos <|ev,e,ve|>); \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   261
\      !!ev1 ev2 ve cl e. \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   262
\        cl = <| ev1, e, ve + {ev2 |-> v_clos(cl)} |> ==> \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   263
\        P ve (fix ev2(ev1) = e) (v_clos cl); \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   264
\      !!ve c1 c2 e1 e2. \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   265
\        [| P ve e1 (v_const c1); P ve e2 (v_const c2) |] ==> \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   266
\        P ve (e1 @ e2) (v_const(c_app c1 c2)); \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   267
\      !!ve vem evm e1 e2 em v v2. \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   268
\        [|  P ve e1 (v_clos <|evm,em,vem|>); \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   269
\            P ve e2 v2; \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   270
\            P (vem + {evm |-> v2}) em v \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   271
\        |] ==> P ve (e1 @ e2) v \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   272
\   |] ==> P ve e v";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   273
by (res_inst_tac [("P","P")] infsys_pp2 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   274
by (rtac eval_ind0 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   275
by (ALLGOALS (rtac infsys_pp1));
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   276
by (ALLGOALS (resolve_tac prems));
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   277
by (REPEAT ((assume_tac 1) ORELSE (dtac infsys_pp2 1)));
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   278
qed "eval_ind";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   279
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   280
(* ############################################################ *)
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   281
(* Elaborations                                                 *)
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   282
(* ############################################################ *)
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   283
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   284
goalw MT.thy [mono_def, elab_fun_def] "mono(elab_fun)";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   285
by infsys_mono_tac;
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   286
qed "elab_fun_mono";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   287
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   288
(* Introduction rules *)
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   289
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   290
val prems = goalw MT.thy [elab_def, elab_rel_def] 
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   291
  "c isof ty ==> te |- e_const(c) ===> ty";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   292
by (cut_facts_tac prems 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   293
by (rtac lfp_intro2 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   294
by (rtac elab_fun_mono 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   295
by (rewtac elab_fun_def);
1820
e381e1c51689 Classical tactics now use default claset.
berghofe
parents: 1584
diff changeset
   296
by (Fast_tac 1);
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   297
qed "elab_const";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   298
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   299
val prems = goalw MT.thy [elab_def, elab_rel_def] 
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   300
  "x:te_dom(te) ==> te |- e_var(x) ===> te_app te x";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   301
by (cut_facts_tac prems 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   302
by (rtac lfp_intro2 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   303
by (rtac elab_fun_mono 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   304
by (rewtac elab_fun_def);
1820
e381e1c51689 Classical tactics now use default claset.
berghofe
parents: 1584
diff changeset
   305
by (Fast_tac 1);
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   306
qed "elab_var";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   307
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   308
val prems = goalw MT.thy [elab_def, elab_rel_def] 
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   309
  "te + {x |=> ty1} |- e ===> ty2 ==> te |- fn x => e ===> ty1->ty2";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   310
by (cut_facts_tac prems 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   311
by (rtac lfp_intro2 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   312
by (rtac elab_fun_mono 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   313
by (rewtac elab_fun_def);
1820
e381e1c51689 Classical tactics now use default claset.
berghofe
parents: 1584
diff changeset
   314
by (Fast_tac 1);
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   315
qed "elab_fn";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   316
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   317
val prems = goalw MT.thy [elab_def, elab_rel_def]
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   318
  " te + {f |=> ty1->ty2} + {x |=> ty1} |- e ===> ty2 ==> \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   319
\   te |- fix f(x) = e ===> ty1->ty2";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   320
by (cut_facts_tac prems 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   321
by (rtac lfp_intro2 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   322
by (rtac elab_fun_mono 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   323
by (rewtac elab_fun_def);
1820
e381e1c51689 Classical tactics now use default claset.
berghofe
parents: 1584
diff changeset
   324
by (Fast_tac 1);
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   325
qed "elab_fix";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   326
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   327
val prems = goalw MT.thy [elab_def, elab_rel_def] 
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   328
  " [| te |- e1 ===> ty1->ty2; te |- e2 ===> ty1 |] ==> \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   329
\   te |- e1 @ e2 ===> ty2";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   330
by (cut_facts_tac prems 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   331
by (rtac lfp_intro2 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   332
by (rtac elab_fun_mono 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   333
by (rewtac elab_fun_def);
1820
e381e1c51689 Classical tactics now use default claset.
berghofe
parents: 1584
diff changeset
   334
by (fast_tac (!claset addSIs [disjI2]) 1);
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   335
qed "elab_app";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   336
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   337
(* Strong elimination, induction on elaborations *)
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   338
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   339
val prems = goalw MT.thy [elab_def, elab_rel_def]
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   340
  " [| te |- e ===> t; \
972
e61b058d58d2 changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents: 969
diff changeset
   341
\      !!te c t. c isof t ==> P(((te,e_const(c)),t)); \
e61b058d58d2 changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents: 969
diff changeset
   342
\      !!te x. x:te_dom(te) ==> P(((te,e_var(x)),te_app te x)); \
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   343
\      !!te x e t1 t2. \
972
e61b058d58d2 changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents: 969
diff changeset
   344
\        [| te + {x |=> t1} |- e ===> t2; P(((te + {x |=> t1},e),t2)) |] ==> \
e61b058d58d2 changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents: 969
diff changeset
   345
\        P(((te,fn x => e),t1->t2)); \
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   346
\      !!te f x e t1 t2. \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   347
\        [| te + {f |=> t1->t2} + {x |=> t1} |- e ===> t2; \
972
e61b058d58d2 changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents: 969
diff changeset
   348
\           P(((te + {f |=> t1->t2} + {x |=> t1},e),t2)) \
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   349
\        |] ==> \
972
e61b058d58d2 changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents: 969
diff changeset
   350
\        P(((te,fix f(x) = e),t1->t2)); \
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   351
\      !!te e1 e2 t1 t2. \
972
e61b058d58d2 changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents: 969
diff changeset
   352
\        [| te |- e1 ===> t1->t2; P(((te,e1),t1->t2)); \
e61b058d58d2 changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents: 969
diff changeset
   353
\           te |- e2 ===> t1; P(((te,e2),t1)) \
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   354
\        |] ==> \
972
e61b058d58d2 changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents: 969
diff changeset
   355
\        P(((te,e1 @ e2),t2)) \
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   356
\   |] ==> \
972
e61b058d58d2 changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents: 969
diff changeset
   357
\   P(((te,e),t))";
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   358
by (resolve_tac (prems RL [lfp_ind2]) 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   359
by (rtac elab_fun_mono 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   360
by (rewtac elab_fun_def);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   361
by (dtac CollectD 1);
1820
e381e1c51689 Classical tactics now use default claset.
berghofe
parents: 1584
diff changeset
   362
by (safe_tac (!claset));
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   363
by (ALLGOALS (resolve_tac prems));
1820
e381e1c51689 Classical tactics now use default claset.
berghofe
parents: 1584
diff changeset
   364
by (ALLGOALS (Fast_tac));
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   365
qed "elab_ind0";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   366
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   367
val prems = goal MT.thy
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   368
  " [| te |- e ===> t; \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   369
\       !!te c t. c isof t ==> P te (e_const c) t; \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   370
\      !!te x. x:te_dom(te) ==> P te (e_var x) (te_app te x); \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   371
\      !!te x e t1 t2. \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   372
\        [| te + {x |=> t1} |- e ===> t2; P (te + {x |=> t1}) e t2 |] ==> \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   373
\        P te (fn x => e) (t1->t2); \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   374
\      !!te f x e t1 t2. \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   375
\        [| te + {f |=> t1->t2} + {x |=> t1} |- e ===> t2; \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   376
\           P (te + {f |=> t1->t2} + {x |=> t1}) e t2 \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   377
\        |] ==> \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   378
\        P te (fix f(x) = e) (t1->t2); \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   379
\      !!te e1 e2 t1 t2. \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   380
\        [| te |- e1 ===> t1->t2; P te e1 (t1->t2); \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   381
\           te |- e2 ===> t1; P te e2 t1 \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   382
\        |] ==> \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   383
\        P te (e1 @ e2) t2 \ 
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   384
\   |] ==> \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   385
\   P te e t";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   386
by (res_inst_tac [("P","P")] infsys_pp2 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   387
by (rtac elab_ind0 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   388
by (ALLGOALS (rtac infsys_pp1));
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   389
by (ALLGOALS (resolve_tac prems));
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   390
by (REPEAT ((assume_tac 1) ORELSE (dtac infsys_pp2 1)));
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   391
qed "elab_ind";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   392
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   393
(* Weak elimination, case analysis on elaborations *)
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   394
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   395
val prems = goalw MT.thy [elab_def, elab_rel_def]
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   396
  " [| te |- e ===> t; \
972
e61b058d58d2 changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents: 969
diff changeset
   397
\      !!te c t. c isof t ==> P(((te,e_const(c)),t)); \
e61b058d58d2 changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents: 969
diff changeset
   398
\      !!te x. x:te_dom(te) ==> P(((te,e_var(x)),te_app te x)); \
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   399
\      !!te x e t1 t2. \
972
e61b058d58d2 changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents: 969
diff changeset
   400
\        te + {x |=> t1} |- e ===> t2 ==> P(((te,fn x => e),t1->t2)); \
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   401
\      !!te f x e t1 t2. \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   402
\        te + {f |=> t1->t2} + {x |=> t1} |- e ===> t2 ==> \
972
e61b058d58d2 changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents: 969
diff changeset
   403
\        P(((te,fix f(x) = e),t1->t2)); \
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   404
\      !!te e1 e2 t1 t2. \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   405
\        [| te |- e1 ===> t1->t2; te |- e2 ===> t1 |] ==> \
972
e61b058d58d2 changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents: 969
diff changeset
   406
\        P(((te,e1 @ e2),t2)) \
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   407
\   |] ==> \
972
e61b058d58d2 changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents: 969
diff changeset
   408
\   P(((te,e),t))";
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   409
by (resolve_tac (prems RL [lfp_elim2]) 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   410
by (rtac elab_fun_mono 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   411
by (rewtac elab_fun_def);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   412
by (dtac CollectD 1);
1820
e381e1c51689 Classical tactics now use default claset.
berghofe
parents: 1584
diff changeset
   413
by (safe_tac (!claset));
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   414
by (ALLGOALS (resolve_tac prems));
1820
e381e1c51689 Classical tactics now use default claset.
berghofe
parents: 1584
diff changeset
   415
by (ALLGOALS (Fast_tac));
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   416
qed "elab_elim0";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   417
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   418
val prems = goal MT.thy
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   419
  " [| te |- e ===> t; \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   420
\       !!te c t. c isof t ==> P te (e_const c) t; \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   421
\      !!te x. x:te_dom(te) ==> P te (e_var x) (te_app te x); \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   422
\      !!te x e t1 t2. \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   423
\        te + {x |=> t1} |- e ===> t2 ==> P te (fn x => e) (t1->t2); \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   424
\      !!te f x e t1 t2. \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   425
\        te + {f |=> t1->t2} + {x |=> t1} |- e ===> t2 ==> \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   426
\        P te (fix f(x) = e) (t1->t2); \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   427
\      !!te e1 e2 t1 t2. \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   428
\        [| te |- e1 ===> t1->t2; te |- e2 ===> t1 |] ==> \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   429
\        P te (e1 @ e2) t2 \ 
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   430
\   |] ==> \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   431
\   P te e t";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   432
by (res_inst_tac [("P","P")] infsys_pp2 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   433
by (rtac elab_elim0 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   434
by (ALLGOALS (rtac infsys_pp1));
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   435
by (ALLGOALS (resolve_tac prems));
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   436
by (REPEAT ((assume_tac 1) ORELSE (dtac infsys_pp2 1)));
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   437
qed "elab_elim";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   438
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   439
(* Elimination rules for each expression *)
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   440
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   441
fun elab_e_elim_tac p = 
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   442
  ( (rtac elab_elim 1) THEN 
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   443
    (resolve_tac p 1) THEN 
1820
e381e1c51689 Classical tactics now use default claset.
berghofe
parents: 1584
diff changeset
   444
    (REPEAT (fast_tac (e_ext_cs (claset_of "HOL")) 1))
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   445
  );
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   446
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   447
val prems = goal MT.thy "te |- e ===> t ==> (e = e_const(c) --> c isof t)";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   448
by (elab_e_elim_tac prems);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   449
qed "elab_const_elim_lem";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   450
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   451
val prems = goal MT.thy "te |- e_const(c) ===> t ==> c isof t";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   452
by (cut_facts_tac prems 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   453
by (dtac elab_const_elim_lem 1);
1820
e381e1c51689 Classical tactics now use default claset.
berghofe
parents: 1584
diff changeset
   454
by (Fast_tac 1);
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   455
qed "elab_const_elim";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   456
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   457
val prems = goal MT.thy 
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   458
  "te |- e ===> t ==> (e = e_var(x) --> t=te_app te x & x:te_dom(te))";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   459
by (elab_e_elim_tac prems);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   460
qed "elab_var_elim_lem";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   461
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   462
val prems = goal MT.thy 
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   463
  "te |- e_var(ev) ===> t ==> t=te_app te ev & ev : te_dom(te)";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   464
by (cut_facts_tac prems 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   465
by (dtac elab_var_elim_lem 1);
1820
e381e1c51689 Classical tactics now use default claset.
berghofe
parents: 1584
diff changeset
   466
by (Fast_tac 1);
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   467
qed "elab_var_elim";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   468
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   469
val prems = goal MT.thy 
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   470
  " te |- e ===> t ==> \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   471
\   ( e = fn x1 => e1 --> \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   472
\     (? t1 t2.t=t_fun t1 t2 & te + {x1 |=> t1} |- e1 ===> t2) \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   473
\   )";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   474
by (elab_e_elim_tac prems);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   475
qed "elab_fn_elim_lem";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   476
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   477
val prems = goal MT.thy 
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   478
  " te |- fn x1 => e1 ===> t ==> \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   479
\   (? t1 t2. t=t1->t2 & te + {x1 |=> t1} |- e1 ===> t2)";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   480
by (cut_facts_tac prems 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   481
by (dtac elab_fn_elim_lem 1);
1820
e381e1c51689 Classical tactics now use default claset.
berghofe
parents: 1584
diff changeset
   482
by (Fast_tac 1);
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   483
qed "elab_fn_elim";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   484
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   485
val prems = goal MT.thy 
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   486
  " te |- e ===> t ==> \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   487
\   (e = fix f(x) = e1 --> \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   488
\   (? t1 t2. t=t1->t2 & te + {f |=> t1->t2} + {x |=> t1} |- e1 ===> t2))"; 
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   489
by (elab_e_elim_tac prems);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   490
qed "elab_fix_elim_lem";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   491
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   492
val prems = goal MT.thy 
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   493
  " te |- fix ev1(ev2) = e1 ===> t ==> \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   494
\   (? t1 t2. t=t1->t2 & te + {ev1 |=> t1->t2} + {ev2 |=> t1} |- e1 ===> t2)";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   495
by (cut_facts_tac prems 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   496
by (dtac elab_fix_elim_lem 1);
1820
e381e1c51689 Classical tactics now use default claset.
berghofe
parents: 1584
diff changeset
   497
by (Fast_tac 1);
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   498
qed "elab_fix_elim";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   499
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   500
val prems = goal MT.thy 
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   501
  " te |- e ===> t2 ==> \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   502
\   (e = e1 @ e2 --> (? t1 . te |- e1 ===> t1->t2 & te |- e2 ===> t1))"; 
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   503
by (elab_e_elim_tac prems);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   504
qed "elab_app_elim_lem";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   505
1266
3ae9fe3c0f68 added local simpsets
clasohm
parents: 1047
diff changeset
   506
val prems = goal MT.thy
3ae9fe3c0f68 added local simpsets
clasohm
parents: 1047
diff changeset
   507
 "te |- e1 @ e2 ===> t2 ==> (? t1 . te |- e1 ===> t1->t2 & te |- e2 ===> t1)"; 
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   508
by (cut_facts_tac prems 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   509
by (dtac elab_app_elim_lem 1);
1820
e381e1c51689 Classical tactics now use default claset.
berghofe
parents: 1584
diff changeset
   510
by (Fast_tac 1);
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   511
qed "elab_app_elim";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   512
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   513
(* ############################################################ *)
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   514
(* The extended correspondence relation                       *)
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   515
(* ############################################################ *)
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   516
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   517
(* Monotonicity of hasty_fun *)
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   518
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   519
goalw MT.thy [mono_def,MT.hasty_fun_def] "mono(hasty_fun)";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   520
by infsys_mono_tac;
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   521
bind_thm("mono_hasty_fun",  result());
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   522
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   523
(* 
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   524
  Because hasty_rel has been defined as the greatest fixpoint of hasty_fun it 
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   525
  enjoys two strong indtroduction (co-induction) rules and an elimination rule.
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   526
*)
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   527
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   528
(* First strong indtroduction (co-induction) rule for hasty_rel *)
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   529
1266
3ae9fe3c0f68 added local simpsets
clasohm
parents: 1047
diff changeset
   530
val prems =
3ae9fe3c0f68 added local simpsets
clasohm
parents: 1047
diff changeset
   531
  goalw MT.thy [hasty_rel_def] "c isof t ==> (v_const(c),t) : hasty_rel";
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   532
by (cut_facts_tac prems 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   533
by (rtac gfp_coind2 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   534
by (rewtac MT.hasty_fun_def);
1047
5133479a37cf Simplified some proofs and made them work for new hyp_subst_tac.
lcp
parents: 972
diff changeset
   535
by (rtac CollectI 1);
5133479a37cf Simplified some proofs and made them work for new hyp_subst_tac.
lcp
parents: 972
diff changeset
   536
by (rtac disjI1 1);
1820
e381e1c51689 Classical tactics now use default claset.
berghofe
parents: 1584
diff changeset
   537
by (Fast_tac 1);
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   538
by (rtac mono_hasty_fun 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   539
qed "hasty_rel_const_coind";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   540
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   541
(* Second strong introduction (co-induction) rule for hasty_rel *)
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   542
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   543
val prems = goalw MT.thy [hasty_rel_def]
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   544
  " [|  te |- fn ev => e ===> t; \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   545
\       ve_dom(ve) = te_dom(te); \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   546
\       ! ev1. \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   547
\         ev1:ve_dom(ve) --> \
972
e61b058d58d2 changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents: 969
diff changeset
   548
\         (ve_app ve ev1,te_app te ev1) : {(v_clos(<|ev,e,ve|>),t)} Un hasty_rel \
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   549
\   |] ==> \
972
e61b058d58d2 changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents: 969
diff changeset
   550
\   (v_clos(<|ev,e,ve|>),t) : hasty_rel";
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   551
by (cut_facts_tac prems 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   552
by (rtac gfp_coind2 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   553
by (rewtac hasty_fun_def);
1047
5133479a37cf Simplified some proofs and made them work for new hyp_subst_tac.
lcp
parents: 972
diff changeset
   554
by (rtac CollectI 1);
5133479a37cf Simplified some proofs and made them work for new hyp_subst_tac.
lcp
parents: 972
diff changeset
   555
by (rtac disjI2 1);
1820
e381e1c51689 Classical tactics now use default claset.
berghofe
parents: 1584
diff changeset
   556
by (fast_tac (claset_of "HOL") 1);
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   557
by (rtac mono_hasty_fun 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   558
qed "hasty_rel_clos_coind";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   559
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   560
(* Elimination rule for hasty_rel *)
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   561
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   562
val prems = goalw MT.thy [hasty_rel_def]
972
e61b058d58d2 changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents: 969
diff changeset
   563
  " [| !! c t.c isof t ==> P((v_const(c),t)); \
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   564
\      !! te ev e t ve. \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   565
\        [| te |- fn ev => e ===> t; \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   566
\           ve_dom(ve) = te_dom(te); \
972
e61b058d58d2 changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents: 969
diff changeset
   567
\           !ev1.ev1:ve_dom(ve) --> (ve_app ve ev1,te_app te ev1) : hasty_rel \
e61b058d58d2 changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents: 969
diff changeset
   568
\        |] ==> P((v_clos(<|ev,e,ve|>),t)); \
e61b058d58d2 changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents: 969
diff changeset
   569
\      (v,t) : hasty_rel \
e61b058d58d2 changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents: 969
diff changeset
   570
\   |] ==> P((v,t))";
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   571
by (cut_facts_tac prems 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   572
by (etac gfp_elim2 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   573
by (rtac mono_hasty_fun 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   574
by (rewtac hasty_fun_def);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   575
by (dtac CollectD 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   576
by (fold_goals_tac [hasty_fun_def]);
1820
e381e1c51689 Classical tactics now use default claset.
berghofe
parents: 1584
diff changeset
   577
by (safe_tac (!claset));
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   578
by (ALLGOALS (resolve_tac prems));
1820
e381e1c51689 Classical tactics now use default claset.
berghofe
parents: 1584
diff changeset
   579
by (ALLGOALS (Fast_tac));
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   580
qed "hasty_rel_elim0";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   581
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   582
val prems = goal MT.thy 
972
e61b058d58d2 changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents: 969
diff changeset
   583
  " [| (v,t) : hasty_rel; \
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   584
\      !! c t.c isof t ==> P (v_const c) t; \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   585
\      !! te ev e t ve. \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   586
\        [| te |- fn ev => e ===> t; \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   587
\           ve_dom(ve) = te_dom(te); \
972
e61b058d58d2 changed syntax of tuples from <..., ...> to (..., ...)
clasohm
parents: 969
diff changeset
   588
\           !ev1.ev1:ve_dom(ve) --> (ve_app ve ev1,te_app te ev1) : hasty_rel \
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   589
\        |] ==> P (v_clos <|ev,e,ve|>) t \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   590
\   |] ==> P v t";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   591
by (res_inst_tac [("P","P")] infsys_p2 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   592
by (rtac hasty_rel_elim0 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   593
by (ALLGOALS (rtac infsys_p1));
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   594
by (ALLGOALS (resolve_tac prems));
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   595
by (REPEAT ((assume_tac 1) ORELSE (dtac infsys_p2 1)));
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   596
qed "hasty_rel_elim";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   597
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   598
(* Introduction rules for hasty *)
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   599
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   600
val prems = goalw MT.thy [hasty_def] "c isof t ==> v_const(c) hasty t";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   601
by (resolve_tac (prems RL [hasty_rel_const_coind]) 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   602
qed "hasty_const";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   603
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   604
val prems = goalw MT.thy [hasty_def,hasty_env_def] 
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   605
  "te |- fn ev => e ===> t & ve hastyenv te ==> v_clos(<|ev,e,ve|>) hasty t";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   606
by (cut_facts_tac prems 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   607
by (rtac hasty_rel_clos_coind 1);
1820
e381e1c51689 Classical tactics now use default claset.
berghofe
parents: 1584
diff changeset
   608
by (ALLGOALS (Fast_tac));
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   609
qed "hasty_clos";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   610
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   611
(* Elimination on constants for hasty *)
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   612
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   613
val prems = goalw MT.thy [hasty_def] 
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   614
  "v hasty t ==> (!c.(v = v_const(c) --> c isof t))";  
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   615
by (cut_facts_tac prems 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   616
by (rtac hasty_rel_elim 1);
1820
e381e1c51689 Classical tactics now use default claset.
berghofe
parents: 1584
diff changeset
   617
by (ALLGOALS (fast_tac (v_ext_cs (claset_of "HOL"))));
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   618
qed "hasty_elim_const_lem";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   619
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   620
val prems = goal MT.thy "v_const(c) hasty t ==> c isof t";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   621
by (cut_facts_tac (prems RL [hasty_elim_const_lem]) 1);
1820
e381e1c51689 Classical tactics now use default claset.
berghofe
parents: 1584
diff changeset
   622
by (Fast_tac 1);
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   623
qed "hasty_elim_const";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   624
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   625
(* Elimination on closures for hasty *)
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   626
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   627
val prems = goalw MT.thy [hasty_env_def,hasty_def] 
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   628
  " v hasty t ==> \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   629
\   ! x e ve. \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   630
\     v=v_clos(<|x,e,ve|>) --> (? te.te |- fn x => e ===> t & ve hastyenv te)";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   631
by (cut_facts_tac prems 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   632
by (rtac hasty_rel_elim 1);
1820
e381e1c51689 Classical tactics now use default claset.
berghofe
parents: 1584
diff changeset
   633
by (ALLGOALS (fast_tac (v_ext_cs (claset_of "HOL"))));
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   634
qed "hasty_elim_clos_lem";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   635
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   636
val prems = goal MT.thy 
1266
3ae9fe3c0f68 added local simpsets
clasohm
parents: 1047
diff changeset
   637
  "v_clos(<|ev,e,ve|>) hasty t ==> ? te.te |- fn ev => e ===>\
3ae9fe3c0f68 added local simpsets
clasohm
parents: 1047
diff changeset
   638
  \t & ve hastyenv te ";
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   639
by (cut_facts_tac (prems RL [hasty_elim_clos_lem]) 1);
1820
e381e1c51689 Classical tactics now use default claset.
berghofe
parents: 1584
diff changeset
   640
by (Fast_tac 1);
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   641
qed "hasty_elim_clos";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   642
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   643
(* ############################################################ *)
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   644
(* The pointwise extension of hasty to environments             *)
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   645
(* ############################################################ *)
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   646
1047
5133479a37cf Simplified some proofs and made them work for new hyp_subst_tac.
lcp
parents: 972
diff changeset
   647
goal MT.thy
5133479a37cf Simplified some proofs and made them work for new hyp_subst_tac.
lcp
parents: 972
diff changeset
   648
  "!!ve. [| ve hastyenv te; v hasty t |] ==> \
5133479a37cf Simplified some proofs and made them work for new hyp_subst_tac.
lcp
parents: 972
diff changeset
   649
\        ve + {ev |-> v} hastyenv te + {ev |=> t}";
5133479a37cf Simplified some proofs and made them work for new hyp_subst_tac.
lcp
parents: 972
diff changeset
   650
by (rewtac hasty_env_def);
1266
3ae9fe3c0f68 added local simpsets
clasohm
parents: 1047
diff changeset
   651
by (asm_full_simp_tac (!simpset delsimps mem_simps
3ae9fe3c0f68 added local simpsets
clasohm
parents: 1047
diff changeset
   652
                                addsimps [ve_dom_owr, te_dom_owr]) 1);
1820
e381e1c51689 Classical tactics now use default claset.
berghofe
parents: 1584
diff changeset
   653
by (safe_tac (claset_of "HOL"));
1047
5133479a37cf Simplified some proofs and made them work for new hyp_subst_tac.
lcp
parents: 972
diff changeset
   654
by (excluded_middle_tac "ev=x" 1);
1266
3ae9fe3c0f68 added local simpsets
clasohm
parents: 1047
diff changeset
   655
by (asm_full_simp_tac (!simpset addsimps [ve_app_owr2, te_app_owr2]) 1);
1820
e381e1c51689 Classical tactics now use default claset.
berghofe
parents: 1584
diff changeset
   656
by (Fast_tac 1);
1266
3ae9fe3c0f68 added local simpsets
clasohm
parents: 1047
diff changeset
   657
by (asm_simp_tac (!simpset addsimps [ve_app_owr1, te_app_owr1]) 1);
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   658
qed "hasty_env1";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   659
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   660
(* ############################################################ *)
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   661
(* The Consistency theorem                                      *)
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   662
(* ############################################################ *)
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   663
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   664
val prems = goal MT.thy 
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   665
  "[| ve hastyenv te ; te |- e_const(c) ===> t |] ==> v_const(c) hasty t";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   666
by (cut_facts_tac prems 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   667
by (dtac elab_const_elim 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   668
by (etac hasty_const 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   669
qed "consistency_const";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   670
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   671
val prems = goalw MT.thy [hasty_env_def]
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   672
  " [| ev : ve_dom(ve); ve hastyenv te ; te |- e_var(ev) ===> t |] ==> \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   673
\   ve_app ve ev hasty t";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   674
by (cut_facts_tac prems 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   675
by (dtac elab_var_elim 1);
1820
e381e1c51689 Classical tactics now use default claset.
berghofe
parents: 1584
diff changeset
   676
by (Fast_tac 1);
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   677
qed "consistency_var";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   678
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   679
val prems = goal MT.thy
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   680
  " [| ve hastyenv te ; te |- fn ev => e ===> t |] ==> \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   681
\   v_clos(<| ev, e, ve |>) hasty t";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   682
by (cut_facts_tac prems 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   683
by (rtac hasty_clos 1);
1820
e381e1c51689 Classical tactics now use default claset.
berghofe
parents: 1584
diff changeset
   684
by (Fast_tac 1);
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   685
qed "consistency_fn";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   686
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   687
val prems = goalw MT.thy [hasty_env_def,hasty_def]
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   688
  " [| cl = <| ev1, e, ve + { ev2 |-> v_clos(cl) } |>; \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   689
\      ve hastyenv te ; \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   690
\      te |- fix ev2  ev1  = e ===> t \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   691
\   |] ==> \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   692
\   v_clos(cl) hasty t";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   693
by (cut_facts_tac prems 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   694
by (dtac elab_fix_elim 1);
1820
e381e1c51689 Classical tactics now use default claset.
berghofe
parents: 1584
diff changeset
   695
by (safe_tac (claset_of "HOL"));
1047
5133479a37cf Simplified some proofs and made them work for new hyp_subst_tac.
lcp
parents: 972
diff changeset
   696
(*Do a single unfolding of cl*)
5133479a37cf Simplified some proofs and made them work for new hyp_subst_tac.
lcp
parents: 972
diff changeset
   697
by ((forward_tac [ssubst] 1) THEN (assume_tac 2));
5133479a37cf Simplified some proofs and made them work for new hyp_subst_tac.
lcp
parents: 972
diff changeset
   698
by (rtac hasty_rel_clos_coind 1);
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   699
by (etac elab_fn 1);
1266
3ae9fe3c0f68 added local simpsets
clasohm
parents: 1047
diff changeset
   700
by (asm_simp_tac (!simpset addsimps [ve_dom_owr, te_dom_owr]) 1);
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   701
1266
3ae9fe3c0f68 added local simpsets
clasohm
parents: 1047
diff changeset
   702
by (asm_simp_tac (!simpset delsimps mem_simps addsimps [ve_dom_owr]) 1);
1820
e381e1c51689 Classical tactics now use default claset.
berghofe
parents: 1584
diff changeset
   703
by (safe_tac (claset_of "HOL"));
1047
5133479a37cf Simplified some proofs and made them work for new hyp_subst_tac.
lcp
parents: 972
diff changeset
   704
by (excluded_middle_tac "ev2=ev1a" 1);
1266
3ae9fe3c0f68 added local simpsets
clasohm
parents: 1047
diff changeset
   705
by (asm_full_simp_tac (!simpset addsimps [ve_app_owr2, te_app_owr2]) 1);
1820
e381e1c51689 Classical tactics now use default claset.
berghofe
parents: 1584
diff changeset
   706
by (Fast_tac 1);
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   707
1266
3ae9fe3c0f68 added local simpsets
clasohm
parents: 1047
diff changeset
   708
by (asm_simp_tac (!simpset delsimps mem_simps
3ae9fe3c0f68 added local simpsets
clasohm
parents: 1047
diff changeset
   709
                           addsimps [ve_app_owr1, te_app_owr1]) 1);
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   710
by (hyp_subst_tac 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   711
by (etac subst 1);
1820
e381e1c51689 Classical tactics now use default claset.
berghofe
parents: 1584
diff changeset
   712
by (Fast_tac 1);
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   713
qed "consistency_fix";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   714
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   715
val prems = goal MT.thy 
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   716
  " [| ! t te. ve hastyenv te  --> te |- e1 ===> t --> v_const(c1) hasty t; \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   717
\      ! t te. ve hastyenv te  --> te |- e2 ===> t --> v_const(c2) hasty t; \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   718
\      ve hastyenv te ; te |- e1 @ e2 ===> t \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   719
\   |] ==> \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   720
\   v_const(c_app c1 c2) hasty t";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   721
by (cut_facts_tac prems 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   722
by (dtac elab_app_elim 1);
1820
e381e1c51689 Classical tactics now use default claset.
berghofe
parents: 1584
diff changeset
   723
by (safe_tac (!claset));
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   724
by (rtac hasty_const 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   725
by (rtac isof_app 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   726
by (rtac hasty_elim_const 1);
1820
e381e1c51689 Classical tactics now use default claset.
berghofe
parents: 1584
diff changeset
   727
by (Fast_tac 1);
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   728
by (rtac hasty_elim_const 1);
1820
e381e1c51689 Classical tactics now use default claset.
berghofe
parents: 1584
diff changeset
   729
by (Fast_tac 1);
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   730
qed "consistency_app1";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   731
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   732
val prems = goal MT.thy 
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   733
  " [| ! t te. \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   734
\        ve hastyenv te  --> \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   735
\        te |- e1 ===> t --> v_clos(<|evm, em, vem|>) hasty t; \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   736
\      ! t te. ve hastyenv te  --> te |- e2 ===> t --> v2 hasty t; \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   737
\      ! t te. \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   738
\        vem + { evm |-> v2 } hastyenv te  --> te |- em ===> t --> v hasty t; \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   739
\      ve hastyenv te ; \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   740
\      te |- e1 @ e2 ===> t \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   741
\   |] ==> \
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   742
\   v hasty t";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   743
by (cut_facts_tac prems 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   744
by (dtac elab_app_elim 1);
1820
e381e1c51689 Classical tactics now use default claset.
berghofe
parents: 1584
diff changeset
   745
by (safe_tac (!claset));
1047
5133479a37cf Simplified some proofs and made them work for new hyp_subst_tac.
lcp
parents: 972
diff changeset
   746
by ((etac allE 1) THEN (etac allE 1) THEN (etac impE 1));
5133479a37cf Simplified some proofs and made them work for new hyp_subst_tac.
lcp
parents: 972
diff changeset
   747
by (assume_tac 1);
5133479a37cf Simplified some proofs and made them work for new hyp_subst_tac.
lcp
parents: 972
diff changeset
   748
by (etac impE 1);
5133479a37cf Simplified some proofs and made them work for new hyp_subst_tac.
lcp
parents: 972
diff changeset
   749
by (assume_tac 1);
5133479a37cf Simplified some proofs and made them work for new hyp_subst_tac.
lcp
parents: 972
diff changeset
   750
by ((etac allE 1) THEN (etac allE 1) THEN (etac impE 1));
5133479a37cf Simplified some proofs and made them work for new hyp_subst_tac.
lcp
parents: 972
diff changeset
   751
by (assume_tac 1);
5133479a37cf Simplified some proofs and made them work for new hyp_subst_tac.
lcp
parents: 972
diff changeset
   752
by (etac impE 1);
5133479a37cf Simplified some proofs and made them work for new hyp_subst_tac.
lcp
parents: 972
diff changeset
   753
by (assume_tac 1);
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   754
by (dtac hasty_elim_clos 1);
1820
e381e1c51689 Classical tactics now use default claset.
berghofe
parents: 1584
diff changeset
   755
by (safe_tac (!claset));
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   756
by (dtac elab_fn_elim 1);
1820
e381e1c51689 Classical tactics now use default claset.
berghofe
parents: 1584
diff changeset
   757
by (safe_tac (!claset));
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   758
by (dtac t_fun_inj 1);
1820
e381e1c51689 Classical tactics now use default claset.
berghofe
parents: 1584
diff changeset
   759
by (safe_tac (!claset));
e381e1c51689 Classical tactics now use default claset.
berghofe
parents: 1584
diff changeset
   760
by ((dtac hasty_env1 1) THEN (assume_tac 1) THEN (Fast_tac 1));
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   761
qed "consistency_app2";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   762
1047
5133479a37cf Simplified some proofs and made them work for new hyp_subst_tac.
lcp
parents: 972
diff changeset
   763
val [major] = goal MT.thy 
5133479a37cf Simplified some proofs and made them work for new hyp_subst_tac.
lcp
parents: 972
diff changeset
   764
  "ve |- e ---> v ==> \
5133479a37cf Simplified some proofs and made them work for new hyp_subst_tac.
lcp
parents: 972
diff changeset
   765
\  (! t te. ve hastyenv te --> te |- e ===> t --> v hasty t)";
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   766
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   767
(* Proof by induction on the structure of evaluations *)
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   768
1047
5133479a37cf Simplified some proofs and made them work for new hyp_subst_tac.
lcp
parents: 972
diff changeset
   769
by (rtac (major RS eval_ind) 1);
1820
e381e1c51689 Classical tactics now use default claset.
berghofe
parents: 1584
diff changeset
   770
by (safe_tac (!claset));
1047
5133479a37cf Simplified some proofs and made them work for new hyp_subst_tac.
lcp
parents: 972
diff changeset
   771
by (DEPTH_SOLVE 
5133479a37cf Simplified some proofs and made them work for new hyp_subst_tac.
lcp
parents: 972
diff changeset
   772
    (ares_tac [consistency_const, consistency_var, consistency_fn,
1465
5d7a7e439cec expanded tabs
clasohm
parents: 1266
diff changeset
   773
               consistency_fix, consistency_app1, consistency_app2] 1));
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   774
qed "consistency";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   775
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   776
(* ############################################################ *)
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   777
(* The Basic Consistency theorem                                *)
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   778
(* ############################################################ *)
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   779
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   780
val prems = goalw MT.thy [isof_env_def,hasty_env_def] 
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   781
  "ve isofenv te ==> ve hastyenv te";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   782
by (cut_facts_tac prems 1);
1820
e381e1c51689 Classical tactics now use default claset.
berghofe
parents: 1584
diff changeset
   783
by (safe_tac (!claset));
1047
5133479a37cf Simplified some proofs and made them work for new hyp_subst_tac.
lcp
parents: 972
diff changeset
   784
by (etac allE 1);
5133479a37cf Simplified some proofs and made them work for new hyp_subst_tac.
lcp
parents: 972
diff changeset
   785
by (etac impE 1);
5133479a37cf Simplified some proofs and made them work for new hyp_subst_tac.
lcp
parents: 972
diff changeset
   786
by (assume_tac 1);
5133479a37cf Simplified some proofs and made them work for new hyp_subst_tac.
lcp
parents: 972
diff changeset
   787
by (etac exE 1);
5133479a37cf Simplified some proofs and made them work for new hyp_subst_tac.
lcp
parents: 972
diff changeset
   788
by (etac conjE 1);
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   789
by (dtac hasty_const 1);
1266
3ae9fe3c0f68 added local simpsets
clasohm
parents: 1047
diff changeset
   790
by (Asm_simp_tac 1);
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   791
qed "basic_consistency_lem";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   792
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   793
val prems = goal MT.thy
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   794
  "[| ve isofenv te; ve |- e ---> v_const(c); te |- e ===> t |] ==> c isof t";
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   795
by (cut_facts_tac prems 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   796
by (rtac hasty_elim_const 1);
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   797
by (dtac consistency 1);
1820
e381e1c51689 Classical tactics now use default claset.
berghofe
parents: 1584
diff changeset
   798
by (fast_tac (!claset addSIs [basic_consistency_lem]) 1);
969
b051e2fc2e34 converted ex with curried function application
clasohm
parents:
diff changeset
   799
qed "basic_consistency";
1584
3d59c407bd36 Sets a lower value of Unify.search_bound
paulson
parents: 1465
diff changeset
   800
3d59c407bd36 Sets a lower value of Unify.search_bound
paulson
parents: 1465
diff changeset
   801
3d59c407bd36 Sets a lower value of Unify.search_bound
paulson
parents: 1465
diff changeset
   802
Unify.search_bound := orig_search_bound;
3d59c407bd36 Sets a lower value of Unify.search_bound
paulson
parents: 1465
diff changeset
   803
3d59c407bd36 Sets a lower value of Unify.search_bound
paulson
parents: 1465
diff changeset
   804
writeln"Reached end of file.";