src/HOL/W0/W.ML
author paulson
Wed, 15 Jul 1998 14:19:02 +0200
changeset 5148 74919e8f221c
parent 5069 3ea049f7979d
child 5184 9b8547a9496a
permissions -rw-r--r--
More tidying and removal of "\!\!... from Goal commands
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
2520
aecaa76e7eff Incorporated Larry's changes.
nipkow
parents: 2518
diff changeset
     1
(* Title:     HOL/W0/W.ML
2518
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
     2
   ID:        $Id$
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
     3
   Author:    Dieter Nazareth and Tobias Nipkow
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
     4
   Copyright  1995 TU Muenchen
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
     5
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
     6
Correctness and completeness of type inference algorithm W
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
     7
*)
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
     8
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
     9
Addsimps [Suc_le_lessD];
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
    10
Delsimps (ex_simps @ all_simps);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
    11
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
    12
(* correctness of W with respect to has_type *)
5148
74919e8f221c More tidying and removal of "\!\!... from Goal commands
paulson
parents: 5069
diff changeset
    13
Goal "!a s t m n . Ok (s,t,m) = W e a n --> $s a |- e :: t";
2518
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
    14
by (expr.induct_tac "e" 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
    15
(* case Var n *)
4686
74a12e86b20b Removed `addsplits [expand_if]'
nipkow
parents: 4089
diff changeset
    16
by (Asm_simp_tac 1);
2518
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
    17
(* case Abs e *)
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4033
diff changeset
    18
by (asm_full_simp_tac (simpset() addsimps [app_subst_list]
4831
dae4d63a1318 Renamed expand_const -> split_const.
nipkow
parents: 4724
diff changeset
    19
                        addsplits [split_bind]) 1);
2518
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
    20
by (strip_tac 1);
3018
e65b60b28341 Ran expandshort
paulson
parents: 3008
diff changeset
    21
by (dtac sym 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4033
diff changeset
    22
by (fast_tac (HOL_cs addss simpset()) 1);
2518
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
    23
(* case App e1 e2 *)
4831
dae4d63a1318 Renamed expand_const -> split_const.
nipkow
parents: 4724
diff changeset
    24
by (simp_tac (simpset() addsplits [split_bind]) 1);
2518
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
    25
by (strip_tac 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
    26
by ( rename_tac "sa ta na sb tb nb sc" 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
    27
by (res_inst_tac [("t2.0","$ sc tb")] has_type.AppI 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
    28
by (res_inst_tac [("s1","sc")] (app_subst_TVar RS subst) 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
    29
by (rtac (app_subst_Fun RS subst) 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
    30
by (res_inst_tac [("t","$sc(tb -> (TVar nb))"),("s","$sc($sb ta)")] subst 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
    31
by (Asm_full_simp_tac 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
    32
by (simp_tac (HOL_ss addsimps [subst_comp_tel RS sym]) 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
    33
by ( (rtac has_type_cl_sub 1) THEN (rtac has_type_cl_sub 1));
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4033
diff changeset
    34
by (asm_full_simp_tac (simpset() addsimps [eq_sym_conv]) 1);
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4033
diff changeset
    35
by (asm_full_simp_tac (simpset() addsimps [subst_comp_tel RS sym,o_def,has_type_cl_sub,eq_sym_conv]) 1);
2518
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
    36
qed_spec_mp "W_correct";
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
    37
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
    38
val has_type_casesE = map(has_type.mk_cases expr.simps)
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
    39
        [" s |- Var n :: t"," s |- Abs e :: t","s |- App e1 e2 ::t"];
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
    40
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
    41
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
    42
(* the resulting type variable is always greater or equal than the given one *)
5148
74919e8f221c More tidying and removal of "\!\!... from Goal commands
paulson
parents: 5069
diff changeset
    43
Goal "!a n s t m. W e a n  = Ok (s,t,m) --> n<=m";
2518
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
    44
by (expr.induct_tac "e" 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
    45
(* case Var(n) *)
4686
74a12e86b20b Removed `addsplits [expand_if]'
nipkow
parents: 4089
diff changeset
    46
by (fast_tac (HOL_cs addss simpset()) 1);
2518
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
    47
(* case Abs e *)
4831
dae4d63a1318 Renamed expand_const -> split_const.
nipkow
parents: 4724
diff changeset
    48
by (simp_tac (simpset() addsplits [split_bind]) 1);
2518
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
    49
by (fast_tac (HOL_cs addDs [Suc_leD]) 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
    50
(* case App e1 e2 *)
4831
dae4d63a1318 Renamed expand_const -> split_const.
nipkow
parents: 4724
diff changeset
    51
by (simp_tac (simpset() addsplits [split_bind]) 1);
2518
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
    52
by (strip_tac 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
    53
by (rename_tac "s t na sa ta nb sb sc tb m" 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
    54
by (eres_inst_tac [("x","a")] allE 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
    55
by (eres_inst_tac [("x","n")] allE 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
    56
by (eres_inst_tac [("x","$ s a")] allE 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
    57
by (eres_inst_tac [("x","s")] allE 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
    58
by (eres_inst_tac [("x","t")] allE 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
    59
by (eres_inst_tac [("x","na")] allE 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
    60
by (eres_inst_tac [("x","na")] allE 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4033
diff changeset
    61
by (asm_full_simp_tac (simpset() addsimps [eq_sym_conv]) 1);
2518
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
    62
by (etac conjE 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
    63
by (eres_inst_tac [("x","sa")] allE 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
    64
by (eres_inst_tac [("x","ta")] allE 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
    65
by (eres_inst_tac [("x","nb")] allE 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
    66
by (res_inst_tac [("j","na")] le_trans 1); 
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
    67
by (Asm_simp_tac 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
    68
by (Asm_simp_tac 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
    69
qed_spec_mp "W_var_ge";
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
    70
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
    71
Addsimps [W_var_ge];
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
    72
5148
74919e8f221c More tidying and removal of "\!\!... from Goal commands
paulson
parents: 5069
diff changeset
    73
Goal "Ok (s,t,m) = W e a n ==> n<=m";
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4033
diff changeset
    74
by (asm_full_simp_tac (simpset() addsimps [eq_sym_conv]) 1);
2518
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
    75
qed "W_var_geD";
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
    76
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
    77
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
    78
(* auxiliary lemma *)
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
    79
goal Maybe.thy "(y = Ok x) = (Ok x = y)";
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4033
diff changeset
    80
by ( simp_tac (simpset() addsimps [eq_sym_conv]) 1);
2518
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
    81
qed "rotate_Ok";
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
    82
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
    83
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
    84
(* resulting type variable is new *)
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4831
diff changeset
    85
Goal
2518
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
    86
     "!n a s t m. new_tv n a --> W e a n = Ok (s,t,m) -->    \
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
    87
\                 new_tv m s & new_tv m t";
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
    88
by (expr.induct_tac "e" 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
    89
(* case Var n *)
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4033
diff changeset
    90
by (fast_tac (HOL_cs addDs [list_all_nth] addss (simpset() 
4686
74a12e86b20b Removed `addsplits [expand_if]'
nipkow
parents: 4089
diff changeset
    91
        addsimps [id_subst_def,new_tv_list,new_tv_subst])) 1);
2518
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
    92
(* case Abs e *)
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4033
diff changeset
    93
by (simp_tac (simpset() addsimps [new_tv_subst,new_tv_Suc_list] 
4831
dae4d63a1318 Renamed expand_const -> split_const.
nipkow
parents: 4724
diff changeset
    94
    addsplits [split_bind]) 1);
2518
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
    95
by (strip_tac 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
    96
by (eres_inst_tac [("x","Suc n")] allE 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
    97
by (eres_inst_tac [("x","(TVar n)#a")] allE 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4033
diff changeset
    98
by (fast_tac (HOL_cs addss (simpset()
2518
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
    99
              addsimps [new_tv_subst,new_tv_Suc_list])) 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   100
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   101
(* case App e1 e2 *)
4831
dae4d63a1318 Renamed expand_const -> split_const.
nipkow
parents: 4724
diff changeset
   102
by (simp_tac (simpset() addsplits [split_bind]) 1);
2518
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   103
by (strip_tac 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   104
by (rename_tac "s t na sa ta nb sb sc tb m" 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   105
by (eres_inst_tac [("x","n")] allE 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   106
by (eres_inst_tac [("x","a")] allE 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   107
by (eres_inst_tac [("x","s")] allE 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   108
by (eres_inst_tac [("x","t")] allE 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   109
by (eres_inst_tac [("x","na")] allE 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   110
by (eres_inst_tac [("x","na")] allE 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4033
diff changeset
   111
by (asm_full_simp_tac (simpset() addsimps [eq_sym_conv]) 1);
2518
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   112
by (eres_inst_tac [("x","$ s a")] allE 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   113
by (eres_inst_tac [("x","sa")] allE 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   114
by (eres_inst_tac [("x","ta")] allE 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   115
by (eres_inst_tac [("x","nb")] allE 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4033
diff changeset
   116
by ( asm_full_simp_tac (simpset() addsimps [o_def,rotate_Ok]) 1);
2518
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   117
by (rtac conjI 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   118
by (rtac new_tv_subst_comp_2 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   119
by (rtac new_tv_subst_comp_2 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   120
by (rtac (lessI RS less_imp_le RS new_tv_subst_le) 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   121
by (res_inst_tac [("n","na")] new_tv_subst_le 1); 
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4033
diff changeset
   122
by (asm_full_simp_tac (simpset() addsimps [rotate_Ok]) 1);
2518
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   123
by (Asm_simp_tac 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   124
by (fast_tac (HOL_cs addDs [W_var_geD] addIs
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   125
     [new_tv_list_le,new_tv_subst_tel,lessI RS less_imp_le RS new_tv_subst_le])
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   126
    1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   127
by (etac (sym RS mgu_new) 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   128
by (best_tac (HOL_cs addDs [W_var_geD] 
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   129
                     addIs [new_tv_subst_te,new_tv_list_le,
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   130
                            new_tv_subst_tel,
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   131
                            lessI RS less_imp_le RS new_tv_le,
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   132
                            lessI RS less_imp_le RS new_tv_subst_le,
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   133
                            new_tv_le]) 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   134
by (fast_tac (HOL_cs addDs [W_var_geD] 
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   135
                     addIs [new_tv_list_le,new_tv_subst_tel,new_tv_le] 
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4033
diff changeset
   136
                     addss (simpset())) 1);
2518
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   137
by (rtac (lessI RS new_tv_subst_var) 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   138
by (etac (sym RS mgu_new) 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   139
by (best_tac (HOL_cs addSIs [lessI RS less_imp_le RS new_tv_le,new_tv_subst_te]
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   140
                     addDs [W_var_geD]
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   141
                     addIs [new_tv_list_le,
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   142
                            new_tv_subst_tel,
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   143
                            lessI RS less_imp_le RS new_tv_subst_le,
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   144
                            new_tv_le] 
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4033
diff changeset
   145
                     addss simpset()) 1);
2518
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   146
by (fast_tac (HOL_cs addDs [W_var_geD] 
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   147
                     addIs [new_tv_list_le,new_tv_subst_tel,new_tv_le]
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4033
diff changeset
   148
                     addss (simpset())) 1);
2518
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   149
qed_spec_mp "new_tv_W";
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   150
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   151
5148
74919e8f221c More tidying and removal of "\!\!... from Goal commands
paulson
parents: 5069
diff changeset
   152
Goal "!n a s t m v. W e a n = Ok (s,t,m) -->            \
2518
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   153
\         (v:free_tv s | v:free_tv t) --> v<n --> v:free_tv a";
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   154
by (expr.induct_tac "e" 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   155
(* case Var n *)
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   156
by (fast_tac (HOL_cs addIs [nth_mem,subsetD,ftv_mem_sub_ftv_list] 
4686
74a12e86b20b Removed `addsplits [expand_if]'
nipkow
parents: 4089
diff changeset
   157
    addss simpset()) 1);
2518
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   158
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   159
(* case Abs e *)
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4033
diff changeset
   160
by (asm_full_simp_tac (simpset() addsimps
4831
dae4d63a1318 Renamed expand_const -> split_const.
nipkow
parents: 4724
diff changeset
   161
    [free_tv_subst] addsplits [split_bind]) 1);
2518
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   162
by (strip_tac 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   163
by (rename_tac "s t na sa ta m v" 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   164
by (eres_inst_tac [("x","Suc n")] allE 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   165
by (eres_inst_tac [("x","TVar n # a")] allE 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   166
by (eres_inst_tac [("x","s")] allE 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   167
by (eres_inst_tac [("x","t")] allE 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   168
by (eres_inst_tac [("x","na")] allE 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   169
by (eres_inst_tac [("x","v")] allE 1);
2520
aecaa76e7eff Incorporated Larry's changes.
nipkow
parents: 2518
diff changeset
   170
by (fast_tac (HOL_cs addSEs [allE]
3008
0a887d5b6718 Ran expandshort
paulson
parents: 2793
diff changeset
   171
                     addIs [cod_app_subst]
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4033
diff changeset
   172
                     addss (simpset() addsimps [less_Suc_eq])) 1);
2520
aecaa76e7eff Incorporated Larry's changes.
nipkow
parents: 2518
diff changeset
   173
(** LEVEL 12 **)
2518
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   174
(* case App e1 e2 *)
4831
dae4d63a1318 Renamed expand_const -> split_const.
nipkow
parents: 4724
diff changeset
   175
by (simp_tac (simpset() addsplits [split_bind]) 1);
2518
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   176
by (strip_tac 1); 
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   177
by (rename_tac "s t na sa ta nb sb sc tb m v" 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   178
by (eres_inst_tac [("x","n")] allE 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   179
by (eres_inst_tac [("x","a")] allE 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   180
by (eres_inst_tac [("x","s")] allE 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   181
by (eres_inst_tac [("x","t")] allE 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   182
by (eres_inst_tac [("x","na")] allE 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   183
by (eres_inst_tac [("x","na")] allE 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   184
by (eres_inst_tac [("x","v")] allE 1);
2520
aecaa76e7eff Incorporated Larry's changes.
nipkow
parents: 2518
diff changeset
   185
(** LEVEL 22 **)
2518
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   186
(* second case *)
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   187
by (eres_inst_tac [("x","$ s a")] allE 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   188
by (eres_inst_tac [("x","sa")] allE 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   189
by (eres_inst_tac [("x","ta")] allE 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   190
by (eres_inst_tac [("x","nb")] allE 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   191
by (eres_inst_tac [("x","v")] allE 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   192
by (safe_tac (empty_cs addSIs [conjI,impI] addSEs [conjE]) ); 
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4033
diff changeset
   193
by (asm_full_simp_tac (simpset() addsimps [rotate_Ok,o_def]) 1);
2518
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   194
by (dtac W_var_geD 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   195
by (dtac W_var_geD 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   196
by ( (forward_tac [less_le_trans] 1) THEN (assume_tac 1) );
2520
aecaa76e7eff Incorporated Larry's changes.
nipkow
parents: 2518
diff changeset
   197
(** LEVEL 32 **)
2518
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   198
by (fast_tac (HOL_cs addDs [free_tv_comp_subst RS subsetD,sym RS mgu_free, 
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   199
    codD,free_tv_app_subst_te RS subsetD,free_tv_app_subst_tel RS subsetD,
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   200
    less_le_trans,less_not_refl2,subsetD]
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   201
  addEs [UnE] 
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4033
diff changeset
   202
  addss simpset()) 1);
2518
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   203
by (Asm_full_simp_tac 1); 
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   204
by (dtac (sym RS W_var_geD) 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   205
by (dtac (sym RS W_var_geD) 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   206
by ( (forward_tac [less_le_trans] 1) THEN (assume_tac 1) );
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   207
by (fast_tac (HOL_cs addDs [mgu_free, codD,free_tv_subst_var RS subsetD,
3008
0a887d5b6718 Ran expandshort
paulson
parents: 2793
diff changeset
   208
                            free_tv_app_subst_te RS subsetD,
0a887d5b6718 Ran expandshort
paulson
parents: 2793
diff changeset
   209
                            free_tv_app_subst_tel RS subsetD,
0a887d5b6718 Ran expandshort
paulson
parents: 2793
diff changeset
   210
                            less_le_trans,subsetD]
0a887d5b6718 Ran expandshort
paulson
parents: 2793
diff changeset
   211
                     addSEs [UnE]
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4033
diff changeset
   212
                     addss simpset()) 1); 
2518
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   213
qed_spec_mp "free_tv_W"; 
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   214
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   215
(* Completeness of W w.r.t. has_type *)
5069
3ea049f7979d isatool fixgoal;
wenzelm
parents: 4831
diff changeset
   216
Goal
2518
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   217
 "!s' a t' n. $s' a |- e :: t' --> new_tv n a -->     \
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   218
\             (? s t. (? m. W e a n = Ok (s,t,m)) &  \
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   219
\                     (? r. $s' a = $r ($s a) & t' = $r t))";
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   220
by (expr.induct_tac "e" 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   221
(* case Var n *)
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   222
by (strip_tac 1);
4686
74a12e86b20b Removed `addsplits [expand_if]'
nipkow
parents: 4089
diff changeset
   223
by (simp_tac (simpset() addcongs [conj_cong]) 1);
2518
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   224
by (eresolve_tac has_type_casesE 1); 
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4033
diff changeset
   225
by (asm_full_simp_tac (simpset() addsimps [eq_sym_conv,app_subst_list]) 1);
2518
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   226
by (res_inst_tac [("x","s'")] exI 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   227
by (Asm_simp_tac 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   228
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   229
(** LEVEL 10 **)
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   230
(* case Abs e *)
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   231
by (strip_tac 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   232
by (eresolve_tac has_type_casesE 1);
3842
b55686a7b22c fixed dots;
wenzelm
parents: 3569
diff changeset
   233
by (eres_inst_tac [("x","%x. if x=n then t1 else (s' x)")] allE 1);
2518
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   234
by (eres_inst_tac [("x","(TVar n)#a")] allE 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   235
by (eres_inst_tac [("x","t2")] allE 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   236
by (eres_inst_tac [("x","Suc n")] allE 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4033
diff changeset
   237
by (fast_tac (HOL_cs addss (simpset() addcongs [conj_cong]
4831
dae4d63a1318 Renamed expand_const -> split_const.
nipkow
parents: 4724
diff changeset
   238
                            addsplits [split_bind])) 1);
2518
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   239
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   240
(** LEVEL 17 **)
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   241
(* case App e1 e2 *)
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   242
by (strip_tac 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   243
by (eresolve_tac has_type_casesE 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   244
by (eres_inst_tac [("x","s'")] allE 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   245
by (eres_inst_tac [("x","a")] allE 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   246
by (eres_inst_tac [("x","t2 -> t'")] allE 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   247
by (eres_inst_tac [("x","n")] allE 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   248
by (safe_tac HOL_cs);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   249
by (eres_inst_tac [("x","r")] allE 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   250
by (eres_inst_tac [("x","$ s a")] allE 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   251
by (eres_inst_tac [("x","t2")] allE 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   252
by (eres_inst_tac [("x","m")] allE 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   253
by (Asm_full_simp_tac 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   254
by (safe_tac HOL_cs);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   255
by (fast_tac (HOL_cs addIs [sym RS W_var_geD,new_tv_W RS
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   256
                            conjunct1,new_tv_list_le,new_tv_subst_tel]) 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   257
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   258
(** LEVEL 35 **)
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   259
by (subgoal_tac
3842
b55686a7b22c fixed dots;
wenzelm
parents: 3569
diff changeset
   260
  "$ (%x. if x=ma then t' else (if x:(free_tv t - free_tv sa) then r x \
2518
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   261
\        else ra x)) ($ sa t) = \
3842
b55686a7b22c fixed dots;
wenzelm
parents: 3569
diff changeset
   262
\  $ (%x. if x=ma then t' else (if x:(free_tv t - free_tv sa) then r x \
2518
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   263
\        else ra x)) (ta -> (TVar ma))" 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   264
by (res_inst_tac [("t","$ (%x. if x = ma then t' else \
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   265
\   (if x:(free_tv t - free_tv sa) then r x else ra x)) ($ sa t)"),
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   266
    ("s","($ ra ta) -> t'")] ssubst 2);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4033
diff changeset
   267
by (asm_simp_tac (simpset() addsimps [subst_comp_te]) 2);
2518
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   268
by (rtac eq_free_eq_subst_te 2);  
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   269
by (strip_tac 2);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   270
by (subgoal_tac "na ~=ma" 2);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   271
by (fast_tac (HOL_cs addDs [new_tv_W,sym RS W_var_geD,
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   272
                            new_tv_not_free_tv,new_tv_le]) 3);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   273
(** LEVEL 42 **)
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   274
by (case_tac "na:free_tv sa" 2);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   275
(* na ~: free_tv sa *)
2793
b30c41754c86 Modified proofs because simplifier does not eta-contract any longer.
nipkow
parents: 2637
diff changeset
   276
by (forward_tac [not_free_impl_id] 3);
4686
74a12e86b20b Removed `addsplits [expand_if]'
nipkow
parents: 4089
diff changeset
   277
by (Asm_simp_tac 3);
2518
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   278
(* na : free_tv sa *)
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   279
by (dres_inst_tac [("ts1","$ s a")] (subst_comp_tel RSN (2,trans)) 2);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   280
by (dtac eq_subst_tel_eq_free 2);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   281
by (fast_tac (HOL_cs addIs [free_tv_W,free_tv_le_new_tv] addDs [new_tv_W]) 2);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   282
by (Asm_simp_tac 2); 
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   283
by (case_tac "na:dom sa" 2);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   284
(* na ~: dom sa *)
2793
b30c41754c86 Modified proofs because simplifier does not eta-contract any longer.
nipkow
parents: 2637
diff changeset
   285
(** LEVEL 50 **)
4686
74a12e86b20b Removed `addsplits [expand_if]'
nipkow
parents: 4089
diff changeset
   286
by (asm_full_simp_tac (simpset() addsimps [dom_def]) 3);
2518
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   287
(* na : dom sa *)
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   288
by (rtac eq_free_eq_subst_te 2);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   289
by (strip_tac 2);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   290
by (subgoal_tac "nb ~= ma" 2);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   291
by ((forward_tac [new_tv_W] 3) THEN (atac 3));
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   292
by (etac conjE 3);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   293
by (dtac new_tv_subst_tel 3);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   294
by (fast_tac (HOL_cs addIs [new_tv_list_le] addDs [sym RS W_var_geD]) 3);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   295
by (fast_tac (set_cs addDs [new_tv_W,new_tv_not_free_tv] addss 
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4033
diff changeset
   296
              (simpset() addsimps [cod_def,free_tv_subst])) 3);
4686
74a12e86b20b Removed `addsplits [expand_if]'
nipkow
parents: 4089
diff changeset
   297
by (fast_tac (set_cs addss (simpset() addsimps [cod_def,free_tv_subst])) 2);
2518
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   298
2793
b30c41754c86 Modified proofs because simplifier does not eta-contract any longer.
nipkow
parents: 2637
diff changeset
   299
(** LEVEL 60 **)
2518
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   300
by (Simp_tac 2);  
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   301
by (rtac eq_free_eq_subst_te 2);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   302
by (strip_tac 2 );
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   303
by (subgoal_tac "na ~= ma" 2);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   304
by ((forward_tac [new_tv_W] 3) THEN (atac 3));
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   305
by (etac conjE 3);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   306
by (dtac (sym RS W_var_geD) 3);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   307
by (fast_tac (HOL_cs addDs [new_tv_list_le,new_tv_subst_tel,new_tv_W,new_tv_not_free_tv]) 3);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   308
by (case_tac "na: free_tv t - free_tv sa" 2);
2793
b30c41754c86 Modified proofs because simplifier does not eta-contract any longer.
nipkow
parents: 2637
diff changeset
   309
(** LEVEL 69 **)
2518
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   310
(* case na ~: free_tv t - free_tv sa *)
4686
74a12e86b20b Removed `addsplits [expand_if]'
nipkow
parents: 4089
diff changeset
   311
by (Asm_full_simp_tac 3);
2518
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   312
(* case na : free_tv t - free_tv sa *)
4686
74a12e86b20b Removed `addsplits [expand_if]'
nipkow
parents: 4089
diff changeset
   313
by (Asm_full_simp_tac 2);
2518
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   314
by (dres_inst_tac [("ts1","$ s a")] (subst_comp_tel RSN (2,trans)) 2);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   315
by (dtac eq_subst_tel_eq_free 2);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   316
by (fast_tac (HOL_cs addIs [free_tv_W,free_tv_le_new_tv] addDs [new_tv_W]) 2);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4033
diff changeset
   317
by (asm_full_simp_tac (simpset() addsimps [free_tv_subst,dom_def]) 2);
2793
b30c41754c86 Modified proofs because simplifier does not eta-contract any longer.
nipkow
parents: 2637
diff changeset
   318
by (Fast_tac 2);
b30c41754c86 Modified proofs because simplifier does not eta-contract any longer.
nipkow
parents: 2637
diff changeset
   319
(** LEVEL 76 **)
4831
dae4d63a1318 Renamed expand_const -> split_const.
nipkow
parents: 4724
diff changeset
   320
by (asm_simp_tac (simpset() addsplits [split_bind]) 1);
2793
b30c41754c86 Modified proofs because simplifier does not eta-contract any longer.
nipkow
parents: 2637
diff changeset
   321
by (safe_tac HOL_cs);
2518
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   322
by (dtac mgu_Ok 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4033
diff changeset
   323
by ( fast_tac (HOL_cs addss simpset()) 1);
2518
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   324
by ((dtac mgu_mg 1) THEN (atac 1));
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   325
by (etac exE 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   326
by (res_inst_tac [("x","rb")] exI 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   327
by (rtac conjI 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   328
by (dres_inst_tac [("x","ma")] fun_cong 2);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4033
diff changeset
   329
by ( asm_full_simp_tac (simpset() addsimps [eq_sym_conv]) 2);
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4033
diff changeset
   330
by (simp_tac (simpset() addsimps [o_def,subst_comp_tel RS sym]) 1);
2793
b30c41754c86 Modified proofs because simplifier does not eta-contract any longer.
nipkow
parents: 2637
diff changeset
   331
(** LEVEL 90 **)
2596
3b4ad6c7726f Modified proofs because of added "triv_forall_equality".
nipkow
parents: 2520
diff changeset
   332
by (rtac ((subst_comp_tel RS sym) RSN (2,trans)) 1);
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4033
diff changeset
   333
by ( asm_full_simp_tac (simpset() addsimps [o_def,eq_sym_conv]) 1);
2518
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   334
by (rtac eq_free_eq_subst_tel 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   335
by ( safe_tac HOL_cs );
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   336
by (subgoal_tac "ma ~= na" 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   337
by ((forward_tac [new_tv_W] 2) THEN (atac 2));
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   338
by (etac conjE 2);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   339
by (dtac new_tv_subst_tel 2);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   340
by (fast_tac (HOL_cs addIs [new_tv_list_le] addDs [sym RS W_var_geD]) 2);
2793
b30c41754c86 Modified proofs because simplifier does not eta-contract any longer.
nipkow
parents: 2637
diff changeset
   341
by (forw_inst_tac [("n","m")] new_tv_W 2 THEN atac 2);
b30c41754c86 Modified proofs because simplifier does not eta-contract any longer.
nipkow
parents: 2637
diff changeset
   342
(** LEVEL 100 **)
2518
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   343
by (etac conjE 2);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   344
by (dtac (free_tv_app_subst_tel RS subsetD) 2);
2793
b30c41754c86 Modified proofs because simplifier does not eta-contract any longer.
nipkow
parents: 2637
diff changeset
   345
by (fast_tac (set_cs addDs [sym RS W_var_geD,new_tv_list_le,codD,
2518
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   346
    new_tv_not_free_tv]) 2);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   347
by (case_tac "na: free_tv t - free_tv sa" 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   348
(* case na ~: free_tv t - free_tv sa *)
4686
74a12e86b20b Removed `addsplits [expand_if]'
nipkow
parents: 4089
diff changeset
   349
by (Asm_full_simp_tac 2);
2518
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   350
(* case na : free_tv t - free_tv sa *)
4686
74a12e86b20b Removed `addsplits [expand_if]'
nipkow
parents: 4089
diff changeset
   351
by (Asm_full_simp_tac 1);
2518
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   352
by (dtac (free_tv_app_subst_tel RS subsetD) 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   353
by (fast_tac (set_cs addDs [codD,subst_comp_tel RSN (2,trans),
3008
0a887d5b6718 Ran expandshort
paulson
parents: 2793
diff changeset
   354
                            eq_subst_tel_eq_free] 
4089
96fba19bcbe2 isatool fixclasimp;
wenzelm
parents: 4033
diff changeset
   355
       addss ((simpset() addsimps [free_tv_subst,dom_def]))) 1);
2518
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   356
(** LEVEL 106 **)
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   357
by (Fast_tac 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   358
qed_spec_mp "W_complete_lemma";
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   359
5148
74919e8f221c More tidying and removal of "\!\!... from Goal commands
paulson
parents: 5069
diff changeset
   360
Goal "[] |- e :: t' ==>  (? s t. (? m. W e [] n = Ok(s,t,m)) &  \
2518
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   361
\                                 (? r. t' = $r t))";
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   362
by (cut_inst_tac [("a","[]"),("s'","id_subst"),("e","e"),("t'","t'")]
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   363
                W_complete_lemma 1);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   364
by (ALLGOALS Asm_full_simp_tac);
bee082efaa46 This is the old version og MiniML for the monomorphic case.
nipkow
parents:
diff changeset
   365
qed "W_complete";