src/HOL/MiniML/Generalize.ML
author nipkow
Fri, 17 Jan 1997 18:50:04 +0100
changeset 2525 477c05586286
child 3018 e65b60b28341
permissions -rw-r--r--
The new version of MiniML including "let".
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
2525
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
     1
(* Title:     HOL/MiniML/Generalize.ML
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
     2
   ID:        $Id$
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
     3
   Author:    Wolfgang Naraschewski and Tobias Nipkow
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
     4
   Copyright  1996 TU Muenchen
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
     5
*)
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
     6
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
     7
AddSEs [equalityE];
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
     8
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
     9
goal thy "!!A B. free_tv A = free_tv B ==> gen A t = gen B t";
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    10
by (typ.induct_tac "t" 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    11
by (ALLGOALS Asm_simp_tac);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    12
qed "gen_eq_on_free_tv";
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    13
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    14
goal thy "!!t.(free_tv t) <= (free_tv sch) --> gen sch t = (mk_scheme t)";
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    15
by (typ.induct_tac "t" 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    16
by (Asm_simp_tac 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    17
by (Simp_tac 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    18
by (Fast_tac 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    19
qed_spec_mp "gen_without_effect";
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    20
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    21
Addsimps [gen_without_effect];
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    22
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    23
goal thy "!!A. free_tv (gen ($ S A) t) = free_tv t Int free_tv ($ S A)";
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    24
by (typ.induct_tac "t" 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    25
by (Simp_tac 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    26
by (case_tac "nat : free_tv ($ S A)" 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    27
by (Asm_simp_tac 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    28
by (Fast_tac 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    29
by (Asm_simp_tac 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    30
by (Fast_tac 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    31
by (Asm_full_simp_tac 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    32
by (Fast_tac 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    33
qed "free_tv_gen";
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    34
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    35
Addsimps [free_tv_gen];
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    36
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    37
goal thy "!!A. free_tv (gen ($ S A) t # $ S A) = free_tv ($ S A)";
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    38
by (Simp_tac 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    39
by (Fast_tac 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    40
qed "free_tv_gen_cons";
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    41
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    42
Addsimps [free_tv_gen_cons];
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    43
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    44
goal thy "!!A. bound_tv (gen A t1) = (free_tv t1) - (free_tv A)";
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    45
by (typ.induct_tac "t1" 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    46
by (Simp_tac 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    47
by (case_tac "nat : free_tv A" 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    48
by (asm_simp_tac (!simpset setloop (split_tac [expand_if])) 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    49
by (asm_simp_tac (!simpset setloop (split_tac [expand_if])) 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    50
by (Fast_tac 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    51
by (Asm_simp_tac 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    52
by (Fast_tac 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    53
qed "bound_tv_gen";
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    54
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    55
Addsimps [bound_tv_gen];
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    56
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    57
goal thy "!!A. new_tv n t --> new_tv n (gen A t)";
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    58
by (typ.induct_tac "t" 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    59
by (Simp_tac 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    60
by (case_tac "nat : free_tv A" 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    61
by (Asm_simp_tac 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    62
by (Asm_simp_tac 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    63
by (Asm_full_simp_tac 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    64
qed_spec_mp "new_tv_compatible_gen";
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    65
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    66
goalw thy [gen_ML_def] "!!A. gen A t = gen_ML A t";
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    67
by (typ.induct_tac "t" 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    68
by (simp_tac (!simpset addsimps [free_tv_ML_scheme_list]) 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    69
by (asm_simp_tac (!simpset addsimps [free_tv_ML_scheme_list]) 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    70
qed "gen_eq_gen_ML";
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    71
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    72
goal thy "!!S. (free_tv S) Int ((free_tv t) - (free_tv A)) = {} \
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    73
\          --> gen ($ S A) ($ S t) = $ S (gen A t)";
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    74
by (typ.induct_tac "t" 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    75
by (strip_tac 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    76
by (case_tac "nat:(free_tv A)" 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    77
by (Asm_simp_tac 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    78
by (Asm_full_simp_tac 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    79
by (subgoal_tac "nat ~: free_tv S" 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    80
by (Fast_tac 2);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    81
by (asm_full_simp_tac (!simpset addsimps [free_tv_subst,dom_def,de_Morgan_disj]) 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    82
by (split_tac [expand_if] 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    83
by (cut_facts_tac [free_tv_app_subst_scheme_list] 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    84
by (Fast_tac 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    85
by (Asm_simp_tac 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    86
by (Best_tac 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    87
qed_spec_mp "gen_subst_commutes";
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    88
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    89
goal Generalize.thy "free_tv(t::typ) <= free_tv(A) --> bound_typ_inst S (gen A t) = t";
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    90
by(typ.induct_tac "t" 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    91
by(ALLGOALS Asm_simp_tac);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    92
by(Fast_tac 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    93
qed_spec_mp "bound_typ_inst_gen";
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    94
Addsimps [bound_typ_inst_gen];
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    95
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    96
goalw Generalize.thy [le_type_scheme_def,is_bound_typ_instance]
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    97
  "gen ($ S A) ($ S t) <= $ S (gen A t)";
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    98
by(safe_tac (!claset));
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
    99
by(rename_tac "R" 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
   100
by(res_inst_tac [("x", "(%a. bound_typ_inst R (gen ($S A) (S a)))")] exI 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
   101
by(typ.induct_tac "t" 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
   102
 by(simp_tac (!simpset setloop (split_tac[expand_if])) 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
   103
by(Asm_simp_tac 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
   104
qed "gen_bound_typ_instance";
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
   105
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
   106
goalw Generalize.thy [le_type_scheme_def,is_bound_typ_instance]
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
   107
  "!!A B. free_tv B <= free_tv A ==> gen A t <= gen B t";
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
   108
by(safe_tac (!claset));
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
   109
by(rename_tac "S" 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
   110
by(res_inst_tac [("x","%b. if b:free_tv A then TVar b else S b")] exI 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
   111
by (typ.induct_tac "t" 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
   112
 by(asm_simp_tac (!simpset setloop (split_tac[expand_if])) 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
   113
 by(Fast_tac 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
   114
by(Asm_simp_tac 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
   115
qed "free_tv_subset_gen_le";
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
   116
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
   117
goalw thy [le_type_scheme_def,is_bound_typ_instance] 
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
   118
      "!!A. new_tv n A --> gen A t <= gen A ($ (%x. TVar (if x : free_tv A then x else n + x)) t)";
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
   119
by (strip_tac 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
   120
by (etac exE 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
   121
by (hyp_subst_tac 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
   122
by (res_inst_tac [("x","(%x. S (if n <= x then x - n else x))")] exI 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
   123
by (typ.induct_tac "t" 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
   124
by (Simp_tac 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
   125
by (case_tac "nat : free_tv A" 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
   126
by (asm_simp_tac (!simpset setloop (split_tac [expand_if])) 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
   127
by (asm_simp_tac (!simpset setloop (split_tac [expand_if])) 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
   128
by (subgoal_tac "n <= n + nat" 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
   129
by (forw_inst_tac [("t","A")] new_tv_le 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
   130
ba 1;
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
   131
by (dtac new_tv_not_free_tv 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
   132
by (dtac new_tv_not_free_tv 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
   133
by (asm_simp_tac (!simpset addsimps [diff_add_inverse]) 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
   134
by (simp_tac (!simpset addsimps [le_add1]) 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
   135
by (Asm_simp_tac 1);
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
   136
qed_spec_mp "gen_t_le_gen_alpha_t";
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
   137
477c05586286 The new version of MiniML including "let".
nipkow
parents:
diff changeset
   138
Addsimps [gen_t_le_gen_alpha_t];