src/ZF/Tools/typechk.ML
author wenzelm
Sun, 15 Mar 2009 20:25:58 +0100
changeset 30541 9f168bdc468a
parent 30528 7173bf123335
child 30722 623d4831c8cf
permissions -rw-r--r--
simplified method setup;
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
12189
4729bbf86626 Isar attribute and method setup;
wenzelm
parents: 12109
diff changeset
     1
(*  Title:      ZF/Tools/typechk.ML
6049
7fef0169ab5e moved from ZF to new subdirectory Tools
paulson
parents:
diff changeset
     2
    Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
6153
bff90585cce5 new typechecking solver for the simplifier
paulson
parents: 6112
diff changeset
     3
    Copyright   1999  University of Cambridge
6049
7fef0169ab5e moved from ZF to new subdirectory Tools
paulson
parents:
diff changeset
     4
18736
541d04c79e12 simplified type attribute;
wenzelm
parents: 18708
diff changeset
     5
Automated type checking (cf. CTT).
6049
7fef0169ab5e moved from ZF to new subdirectory Tools
paulson
parents:
diff changeset
     6
*)
7fef0169ab5e moved from ZF to new subdirectory Tools
paulson
parents:
diff changeset
     7
12189
4729bbf86626 Isar attribute and method setup;
wenzelm
parents: 12109
diff changeset
     8
signature TYPE_CHECK =
4729bbf86626 Isar attribute and method setup;
wenzelm
parents: 12109
diff changeset
     9
sig
21506
b2a673894ce5 prefer Proof.context over Context.generic;
wenzelm
parents: 20193
diff changeset
    10
  val print_tcset: Proof.context -> unit
18736
541d04c79e12 simplified type attribute;
wenzelm
parents: 18708
diff changeset
    11
  val TC_add: attribute
541d04c79e12 simplified type attribute;
wenzelm
parents: 18708
diff changeset
    12
  val TC_del: attribute
541d04c79e12 simplified type attribute;
wenzelm
parents: 18708
diff changeset
    13
  val typecheck_tac: Proof.context -> tactic
541d04c79e12 simplified type attribute;
wenzelm
parents: 18708
diff changeset
    14
  val type_solver_tac: Proof.context -> thm list -> int -> tactic
541d04c79e12 simplified type attribute;
wenzelm
parents: 18708
diff changeset
    15
  val type_solver: solver
18708
4b3dadb4fe33 setup: theory -> theory;
wenzelm
parents: 17886
diff changeset
    16
  val setup: theory -> theory
12189
4729bbf86626 Isar attribute and method setup;
wenzelm
parents: 12109
diff changeset
    17
end;
4729bbf86626 Isar attribute and method setup;
wenzelm
parents: 12109
diff changeset
    18
4729bbf86626 Isar attribute and method setup;
wenzelm
parents: 12109
diff changeset
    19
structure TypeCheck: TYPE_CHECK =
6153
bff90585cce5 new typechecking solver for the simplifier
paulson
parents: 6112
diff changeset
    20
struct
12189
4729bbf86626 Isar attribute and method setup;
wenzelm
parents: 12109
diff changeset
    21
18736
541d04c79e12 simplified type attribute;
wenzelm
parents: 18708
diff changeset
    22
(* datatype tcset *)
541d04c79e12 simplified type attribute;
wenzelm
parents: 18708
diff changeset
    23
541d04c79e12 simplified type attribute;
wenzelm
parents: 18708
diff changeset
    24
datatype tcset = TC of
541d04c79e12 simplified type attribute;
wenzelm
parents: 18708
diff changeset
    25
 {rules: thm list,     (*the type-checking rules*)
541d04c79e12 simplified type attribute;
wenzelm
parents: 18708
diff changeset
    26
  net: thm Net.net};   (*discrimination net of the same rules*)
541d04c79e12 simplified type attribute;
wenzelm
parents: 18708
diff changeset
    27
541d04c79e12 simplified type attribute;
wenzelm
parents: 18708
diff changeset
    28
fun add_rule th (tcs as TC {rules, net}) =
22360
26ead7ed4f4b moved eq_thm etc. to structure Thm in Pure/more_thm.ML;
wenzelm
parents: 21506
diff changeset
    29
  if member Thm.eq_thm_prop rules th then
18736
541d04c79e12 simplified type attribute;
wenzelm
parents: 18708
diff changeset
    30
    (warning ("Ignoring duplicate type-checking rule\n" ^ Display.string_of_thm th); tcs)
541d04c79e12 simplified type attribute;
wenzelm
parents: 18708
diff changeset
    31
  else
541d04c79e12 simplified type attribute;
wenzelm
parents: 18708
diff changeset
    32
    TC {rules = th :: rules,
541d04c79e12 simplified type attribute;
wenzelm
parents: 18708
diff changeset
    33
        net = Net.insert_term (K false) (Thm.concl_of th, th) net};
541d04c79e12 simplified type attribute;
wenzelm
parents: 18708
diff changeset
    34
541d04c79e12 simplified type attribute;
wenzelm
parents: 18708
diff changeset
    35
fun del_rule th (tcs as TC {rules, net}) =
22360
26ead7ed4f4b moved eq_thm etc. to structure Thm in Pure/more_thm.ML;
wenzelm
parents: 21506
diff changeset
    36
  if member Thm.eq_thm_prop rules th then
26ead7ed4f4b moved eq_thm etc. to structure Thm in Pure/more_thm.ML;
wenzelm
parents: 21506
diff changeset
    37
    TC {net = Net.delete_term Thm.eq_thm_prop (Thm.concl_of th, th) net,
26ead7ed4f4b moved eq_thm etc. to structure Thm in Pure/more_thm.ML;
wenzelm
parents: 21506
diff changeset
    38
        rules = remove Thm.eq_thm_prop th rules}
18736
541d04c79e12 simplified type attribute;
wenzelm
parents: 18708
diff changeset
    39
  else (warning ("No such type-checking rule\n" ^ Display.string_of_thm th); tcs);
6153
bff90585cce5 new typechecking solver for the simplifier
paulson
parents: 6112
diff changeset
    40
bff90585cce5 new typechecking solver for the simplifier
paulson
parents: 6112
diff changeset
    41
18736
541d04c79e12 simplified type attribute;
wenzelm
parents: 18708
diff changeset
    42
(* generic data *)
541d04c79e12 simplified type attribute;
wenzelm
parents: 18708
diff changeset
    43
541d04c79e12 simplified type attribute;
wenzelm
parents: 18708
diff changeset
    44
structure Data = GenericDataFun
541d04c79e12 simplified type attribute;
wenzelm
parents: 18708
diff changeset
    45
(
541d04c79e12 simplified type attribute;
wenzelm
parents: 18708
diff changeset
    46
  type T = tcset
541d04c79e12 simplified type attribute;
wenzelm
parents: 18708
diff changeset
    47
  val empty = TC {rules = [], net = Net.empty};
541d04c79e12 simplified type attribute;
wenzelm
parents: 18708
diff changeset
    48
  val extend = I;
6153
bff90585cce5 new typechecking solver for the simplifier
paulson
parents: 6112
diff changeset
    49
18736
541d04c79e12 simplified type attribute;
wenzelm
parents: 18708
diff changeset
    50
  fun merge _ (TC {rules, net}, TC {rules = rules', net = net'}) =
24039
273698405054 renamed Drule.add/del/merge_rules to Thm.add/del/merge_thms;
wenzelm
parents: 22846
diff changeset
    51
    TC {rules = Thm.merge_thms (rules, rules'),
22360
26ead7ed4f4b moved eq_thm etc. to structure Thm in Pure/more_thm.ML;
wenzelm
parents: 21506
diff changeset
    52
        net = Net.merge Thm.eq_thm_prop (net, net')};
18736
541d04c79e12 simplified type attribute;
wenzelm
parents: 18708
diff changeset
    53
);
541d04c79e12 simplified type attribute;
wenzelm
parents: 18708
diff changeset
    54
541d04c79e12 simplified type attribute;
wenzelm
parents: 18708
diff changeset
    55
val TC_add = Thm.declaration_attribute (Data.map o add_rule);
541d04c79e12 simplified type attribute;
wenzelm
parents: 18708
diff changeset
    56
val TC_del = Thm.declaration_attribute (Data.map o del_rule);
541d04c79e12 simplified type attribute;
wenzelm
parents: 18708
diff changeset
    57
541d04c79e12 simplified type attribute;
wenzelm
parents: 18708
diff changeset
    58
val tcset_of = Data.get o Context.Proof;
6153
bff90585cce5 new typechecking solver for the simplifier
paulson
parents: 6112
diff changeset
    59
22846
fb79144af9a3 simplified DataFun interfaces;
wenzelm
parents: 22360
diff changeset
    60
fun print_tcset ctxt =
fb79144af9a3 simplified DataFun interfaces;
wenzelm
parents: 22360
diff changeset
    61
  let val TC {rules, ...} = tcset_of ctxt in
fb79144af9a3 simplified DataFun interfaces;
wenzelm
parents: 22360
diff changeset
    62
    Pretty.writeln (Pretty.big_list "type-checking rules:"
fb79144af9a3 simplified DataFun interfaces;
wenzelm
parents: 22360
diff changeset
    63
      (map (ProofContext.pretty_thm ctxt) rules))
fb79144af9a3 simplified DataFun interfaces;
wenzelm
parents: 22360
diff changeset
    64
  end;
fb79144af9a3 simplified DataFun interfaces;
wenzelm
parents: 22360
diff changeset
    65
6153
bff90585cce5 new typechecking solver for the simplifier
paulson
parents: 6112
diff changeset
    66
18736
541d04c79e12 simplified type attribute;
wenzelm
parents: 18708
diff changeset
    67
(* tactics *)
6153
bff90585cce5 new typechecking solver for the simplifier
paulson
parents: 6112
diff changeset
    68
bff90585cce5 new typechecking solver for the simplifier
paulson
parents: 6112
diff changeset
    69
(*resolution using a net rather than rules*)
bff90585cce5 new typechecking solver for the simplifier
paulson
parents: 6112
diff changeset
    70
fun net_res_tac maxr net =
bff90585cce5 new typechecking solver for the simplifier
paulson
parents: 6112
diff changeset
    71
  SUBGOAL
bff90585cce5 new typechecking solver for the simplifier
paulson
parents: 6112
diff changeset
    72
    (fn (prem,i) =>
bff90585cce5 new typechecking solver for the simplifier
paulson
parents: 6112
diff changeset
    73
      let val rls = Net.unify_term net (Logic.strip_assums_concl prem)
12189
4729bbf86626 Isar attribute and method setup;
wenzelm
parents: 12109
diff changeset
    74
      in
4729bbf86626 Isar attribute and method setup;
wenzelm
parents: 12109
diff changeset
    75
         if length rls <= maxr then resolve_tac rls i else no_tac
6153
bff90585cce5 new typechecking solver for the simplifier
paulson
parents: 6112
diff changeset
    76
      end);
bff90585cce5 new typechecking solver for the simplifier
paulson
parents: 6112
diff changeset
    77
24826
78e6a3cea367 avoid unnamed infixes;
wenzelm
parents: 24039
diff changeset
    78
fun is_rigid_elem (Const("Trueprop",_) $ (Const(@{const_name mem},_) $ a $ _)) =
6049
7fef0169ab5e moved from ZF to new subdirectory Tools
paulson
parents:
diff changeset
    79
      not (is_Var (head_of a))
7fef0169ab5e moved from ZF to new subdirectory Tools
paulson
parents:
diff changeset
    80
  | is_rigid_elem _ = false;
7fef0169ab5e moved from ZF to new subdirectory Tools
paulson
parents:
diff changeset
    81
12189
4729bbf86626 Isar attribute and method setup;
wenzelm
parents: 12109
diff changeset
    82
(*Try solving a:A by assumption provided a is rigid!*)
6049
7fef0169ab5e moved from ZF to new subdirectory Tools
paulson
parents:
diff changeset
    83
val test_assume_tac = SUBGOAL(fn (prem,i) =>
7fef0169ab5e moved from ZF to new subdirectory Tools
paulson
parents:
diff changeset
    84
    if is_rigid_elem (Logic.strip_assums_concl prem)
7fef0169ab5e moved from ZF to new subdirectory Tools
paulson
parents:
diff changeset
    85
    then  assume_tac i  else  eq_assume_tac i);
7fef0169ab5e moved from ZF to new subdirectory Tools
paulson
parents:
diff changeset
    86
12189
4729bbf86626 Isar attribute and method setup;
wenzelm
parents: 12109
diff changeset
    87
(*Type checking solves a:?A (a rigid, ?A maybe flexible).
6049
7fef0169ab5e moved from ZF to new subdirectory Tools
paulson
parents:
diff changeset
    88
  match_tac is too strict; would refuse to instantiate ?A*)
6153
bff90585cce5 new typechecking solver for the simplifier
paulson
parents: 6112
diff changeset
    89
fun typecheck_step_tac (TC{net,...}) =
bff90585cce5 new typechecking solver for the simplifier
paulson
parents: 6112
diff changeset
    90
    FIRSTGOAL (test_assume_tac ORELSE' net_res_tac 3 net);
6049
7fef0169ab5e moved from ZF to new subdirectory Tools
paulson
parents:
diff changeset
    91
18736
541d04c79e12 simplified type attribute;
wenzelm
parents: 18708
diff changeset
    92
fun typecheck_tac ctxt = REPEAT (typecheck_step_tac (tcset_of ctxt));
6049
7fef0169ab5e moved from ZF to new subdirectory Tools
paulson
parents:
diff changeset
    93
6153
bff90585cce5 new typechecking solver for the simplifier
paulson
parents: 6112
diff changeset
    94
(*Compiles a term-net for speed*)
26287
df8e5362cff9 proper antiquotations;
wenzelm
parents: 24893
diff changeset
    95
val basic_res_tac = net_resolve_tac [@{thm TrueI}, @{thm refl}, reflexive_thm, @{thm iff_refl},
df8e5362cff9 proper antiquotations;
wenzelm
parents: 24893
diff changeset
    96
                                     @{thm ballI}, @{thm allI}, @{thm conjI}, @{thm impI}];
6049
7fef0169ab5e moved from ZF to new subdirectory Tools
paulson
parents:
diff changeset
    97
7fef0169ab5e moved from ZF to new subdirectory Tools
paulson
parents:
diff changeset
    98
(*Instantiates variables in typing conditions.
7fef0169ab5e moved from ZF to new subdirectory Tools
paulson
parents:
diff changeset
    99
  drawback: does not simplify conjunctions*)
18736
541d04c79e12 simplified type attribute;
wenzelm
parents: 18708
diff changeset
   100
fun type_solver_tac ctxt hyps = SELECT_GOAL
6153
bff90585cce5 new typechecking solver for the simplifier
paulson
parents: 6112
diff changeset
   101
    (DEPTH_SOLVE (etac FalseE 1
12189
4729bbf86626 Isar attribute and method setup;
wenzelm
parents: 12109
diff changeset
   102
                  ORELSE basic_res_tac 1
4729bbf86626 Isar attribute and method setup;
wenzelm
parents: 12109
diff changeset
   103
                  ORELSE (ares_tac hyps 1
18736
541d04c79e12 simplified type attribute;
wenzelm
parents: 18708
diff changeset
   104
                          APPEND typecheck_step_tac (tcset_of ctxt))));
12189
4729bbf86626 Isar attribute and method setup;
wenzelm
parents: 12109
diff changeset
   105
18736
541d04c79e12 simplified type attribute;
wenzelm
parents: 18708
diff changeset
   106
val type_solver = Simplifier.mk_solver' "ZF typecheck" (fn ss =>
541d04c79e12 simplified type attribute;
wenzelm
parents: 18708
diff changeset
   107
  type_solver_tac (Simplifier.the_context ss) (Simplifier.prems_of_ss ss));
6153
bff90585cce5 new typechecking solver for the simplifier
paulson
parents: 6112
diff changeset
   108
bff90585cce5 new typechecking solver for the simplifier
paulson
parents: 6112
diff changeset
   109
18736
541d04c79e12 simplified type attribute;
wenzelm
parents: 18708
diff changeset
   110
(* concrete syntax *)
12189
4729bbf86626 Isar attribute and method setup;
wenzelm
parents: 12109
diff changeset
   111
18736
541d04c79e12 simplified type attribute;
wenzelm
parents: 18708
diff changeset
   112
val typecheck_meth =
30541
9f168bdc468a simplified method setup;
wenzelm
parents: 30528
diff changeset
   113
  Method.sections
18736
541d04c79e12 simplified type attribute;
wenzelm
parents: 18708
diff changeset
   114
    [Args.add -- Args.colon >> K (I, TC_add),
541d04c79e12 simplified type attribute;
wenzelm
parents: 18708
diff changeset
   115
     Args.del -- Args.colon >> K (I, TC_del)]
30541
9f168bdc468a simplified method setup;
wenzelm
parents: 30528
diff changeset
   116
  >> (K (fn ctxt => SIMPLE_METHOD (CHANGED (typecheck_tac ctxt))));
12189
4729bbf86626 Isar attribute and method setup;
wenzelm
parents: 12109
diff changeset
   117
24867
e5b55d7be9bb simplified interfaces for outer syntax;
wenzelm
parents: 24826
diff changeset
   118
val _ =
e5b55d7be9bb simplified interfaces for outer syntax;
wenzelm
parents: 24826
diff changeset
   119
  OuterSyntax.improper_command "print_tcset" "print context of ZF typecheck" OuterKeyword.diag
18736
541d04c79e12 simplified type attribute;
wenzelm
parents: 18708
diff changeset
   120
    (Scan.succeed (Toplevel.no_timing o Toplevel.unknown_context o
24867
e5b55d7be9bb simplified interfaces for outer syntax;
wenzelm
parents: 24826
diff changeset
   121
      Toplevel.keep (print_tcset o Toplevel.context_of)));
12189
4729bbf86626 Isar attribute and method setup;
wenzelm
parents: 12109
diff changeset
   122
4729bbf86626 Isar attribute and method setup;
wenzelm
parents: 12109
diff changeset
   123
18736
541d04c79e12 simplified type attribute;
wenzelm
parents: 18708
diff changeset
   124
(* theory setup *)
12189
4729bbf86626 Isar attribute and method setup;
wenzelm
parents: 12109
diff changeset
   125
4729bbf86626 Isar attribute and method setup;
wenzelm
parents: 12109
diff changeset
   126
val setup =
30528
7173bf123335 simplified attribute setup;
wenzelm
parents: 30510
diff changeset
   127
  Attrib.setup @{binding TC} (Attrib.add_del TC_add TC_del) "declaration of type-checking rule" #>
30541
9f168bdc468a simplified method setup;
wenzelm
parents: 30528
diff changeset
   128
  Method.setup @{binding typecheck} typecheck_meth "ZF type-checking" #>
26496
49ae9456eba9 purely functional setup of claset/simpset/clasimpset;
wenzelm
parents: 26287
diff changeset
   129
  Simplifier.map_simpset (fn ss => ss setSolver type_solver);
12189
4729bbf86626 Isar attribute and method setup;
wenzelm
parents: 12109
diff changeset
   130
4729bbf86626 Isar attribute and method setup;
wenzelm
parents: 12109
diff changeset
   131
end;