TFL/post.sml
author paulson
Thu, 01 Oct 1998 18:30:05 +0200
changeset 5601 b6456ccd9e3e
parent 5103 866a281a8c2a
child 5962 0f7375e5e977
permissions -rw-r--r--
revised for new treatment of integers
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
3302
404fe31fd8d2 New headers and other minor changes
paulson
parents: 3271
diff changeset
     1
(*  Title:      TFL/post
404fe31fd8d2 New headers and other minor changes
paulson
parents: 3271
diff changeset
     2
    ID:         $Id$
404fe31fd8d2 New headers and other minor changes
paulson
parents: 3271
diff changeset
     3
    Author:     Konrad Slind, Cambridge University Computer Laboratory
404fe31fd8d2 New headers and other minor changes
paulson
parents: 3271
diff changeset
     4
    Copyright   1997  University of Cambridge
404fe31fd8d2 New headers and other minor changes
paulson
parents: 3271
diff changeset
     5
404fe31fd8d2 New headers and other minor changes
paulson
parents: 3271
diff changeset
     6
Postprocessing of TFL definitions
404fe31fd8d2 New headers and other minor changes
paulson
parents: 3271
diff changeset
     7
*)
404fe31fd8d2 New headers and other minor changes
paulson
parents: 3271
diff changeset
     8
3191
14bd6e5985f1 TFL now integrated with HOL (more work needed)
paulson
parents: 2467
diff changeset
     9
signature TFL = 
14bd6e5985f1 TFL now integrated with HOL (more work needed)
paulson
parents: 2467
diff changeset
    10
  sig
2112
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
    11
   structure Prim : TFL_sig
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
    12
3191
14bd6e5985f1 TFL now integrated with HOL (more work needed)
paulson
parents: 2467
diff changeset
    13
   val tgoalw : theory -> thm list -> thm list -> thm list
14bd6e5985f1 TFL now integrated with HOL (more work needed)
paulson
parents: 2467
diff changeset
    14
   val tgoal: theory -> thm list -> thm list
2112
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
    15
3405
2cccd0e3e9ea Numerous simplifications and removal of HOL-isms
paulson
parents: 3391
diff changeset
    16
   val std_postprocessor : simpset -> theory 
2112
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
    17
                           -> {induction:thm, rules:thm, TCs:term list list} 
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
    18
                           -> {induction:thm, rules:thm, nested_tcs:thm list}
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
    19
3927
27c63b757af5 adapted to qualified names;
wenzelm
parents: 3572
diff changeset
    20
   val define_i : theory -> xstring -> term -> term list
3405
2cccd0e3e9ea Numerous simplifications and removal of HOL-isms
paulson
parents: 3391
diff changeset
    21
                  -> theory * Prim.pattern list
3331
c81c7f8ad333 Now checks the name of the function being defined
paulson
parents: 3302
diff changeset
    22
3927
27c63b757af5 adapted to qualified names;
wenzelm
parents: 3572
diff changeset
    23
   val define   : theory -> xstring -> string -> string list 
3331
c81c7f8ad333 Now checks the name of the function being defined
paulson
parents: 3302
diff changeset
    24
                  -> theory * Prim.pattern list
2112
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
    25
3459
112cbb8301dc Removal of structure Context and its replacement by a theorem list of
paulson
parents: 3405
diff changeset
    26
   val simplify_defn : simpset * thm list 
112cbb8301dc Removal of structure Context and its replacement by a theorem list of
paulson
parents: 3405
diff changeset
    27
                        -> theory * (string * Prim.pattern list)
3191
14bd6e5985f1 TFL now integrated with HOL (more work needed)
paulson
parents: 2467
diff changeset
    28
                        -> {rules:thm list, induct:thm, tcs:term list}
2112
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
    29
3191
14bd6e5985f1 TFL now integrated with HOL (more work needed)
paulson
parents: 2467
diff changeset
    30
  (*-------------------------------------------------------------------------
14bd6e5985f1 TFL now integrated with HOL (more work needed)
paulson
parents: 2467
diff changeset
    31
       val function : theory -> term -> {theory:theory, eq_ind : thm}
14bd6e5985f1 TFL now integrated with HOL (more work needed)
paulson
parents: 2467
diff changeset
    32
       val lazyR_def: theory -> term -> {theory:theory, eqns : thm}
14bd6e5985f1 TFL now integrated with HOL (more work needed)
paulson
parents: 2467
diff changeset
    33
   *-------------------------------------------------------------------------*)
2112
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
    34
3191
14bd6e5985f1 TFL now integrated with HOL (more work needed)
paulson
parents: 2467
diff changeset
    35
  end;
14bd6e5985f1 TFL now integrated with HOL (more work needed)
paulson
parents: 2467
diff changeset
    36
14bd6e5985f1 TFL now integrated with HOL (more work needed)
paulson
parents: 2467
diff changeset
    37
14bd6e5985f1 TFL now integrated with HOL (more work needed)
paulson
parents: 2467
diff changeset
    38
structure Tfl: TFL =
2112
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
    39
struct
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
    40
 structure Prim = Prim
3391
5e45dd3b64e9 More de-HOLification: using Free, Const, etc. instead of mk_var, mk_const
paulson
parents: 3331
diff changeset
    41
 structure S = USyntax
2112
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
    42
3191
14bd6e5985f1 TFL now integrated with HOL (more work needed)
paulson
parents: 2467
diff changeset
    43
(*---------------------------------------------------------------------------
14bd6e5985f1 TFL now integrated with HOL (more work needed)
paulson
parents: 2467
diff changeset
    44
 * Extract termination goals so that they can be put it into a goalstack, or 
14bd6e5985f1 TFL now integrated with HOL (more work needed)
paulson
parents: 2467
diff changeset
    45
 * have a tactic directly applied to them.
14bd6e5985f1 TFL now integrated with HOL (more work needed)
paulson
parents: 2467
diff changeset
    46
 *--------------------------------------------------------------------------*)
14bd6e5985f1 TFL now integrated with HOL (more work needed)
paulson
parents: 2467
diff changeset
    47
fun termination_goals rules = 
3405
2cccd0e3e9ea Numerous simplifications and removal of HOL-isms
paulson
parents: 3391
diff changeset
    48
    map (#1 o Type.freeze_thaw o HOLogic.dest_Trueprop)
3191
14bd6e5985f1 TFL now integrated with HOL (more work needed)
paulson
parents: 2467
diff changeset
    49
      (foldr (fn (th,A) => union_term (prems_of th, A)) (rules, []));
14bd6e5985f1 TFL now integrated with HOL (more work needed)
paulson
parents: 2467
diff changeset
    50
3405
2cccd0e3e9ea Numerous simplifications and removal of HOL-isms
paulson
parents: 3391
diff changeset
    51
(*---------------------------------------------------------------------------
2cccd0e3e9ea Numerous simplifications and removal of HOL-isms
paulson
parents: 3391
diff changeset
    52
 * Finds the termination conditions in (highly massaged) definition and 
2cccd0e3e9ea Numerous simplifications and removal of HOL-isms
paulson
parents: 3391
diff changeset
    53
 * puts them into a goalstack.
2cccd0e3e9ea Numerous simplifications and removal of HOL-isms
paulson
parents: 3391
diff changeset
    54
 *--------------------------------------------------------------------------*)
2cccd0e3e9ea Numerous simplifications and removal of HOL-isms
paulson
parents: 3391
diff changeset
    55
fun tgoalw thy defs rules = 
3497
122e80826c95 Now catches the error of calling tgoalw when there are no goals to prove,
paulson
parents: 3459
diff changeset
    56
  case termination_goals rules of
122e80826c95 Now catches the error of calling tgoalw when there are no goals to prove,
paulson
parents: 3459
diff changeset
    57
      [] => error "tgoalw: no termination conditions to prove"
122e80826c95 Now catches the error of calling tgoalw when there are no goals to prove,
paulson
parents: 3459
diff changeset
    58
    | L  => goalw_cterm defs 
122e80826c95 Now catches the error of calling tgoalw when there are no goals to prove,
paulson
parents: 3459
diff changeset
    59
              (cterm_of (sign_of thy) 
122e80826c95 Now catches the error of calling tgoalw when there are no goals to prove,
paulson
parents: 3459
diff changeset
    60
	                (HOLogic.mk_Trueprop(USyntax.list_mk_conj L)));
2112
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
    61
3405
2cccd0e3e9ea Numerous simplifications and removal of HOL-isms
paulson
parents: 3391
diff changeset
    62
fun tgoal thy = tgoalw thy [];
2112
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
    63
3405
2cccd0e3e9ea Numerous simplifications and removal of HOL-isms
paulson
parents: 3391
diff changeset
    64
(*---------------------------------------------------------------------------
2cccd0e3e9ea Numerous simplifications and removal of HOL-isms
paulson
parents: 3391
diff changeset
    65
* Three postprocessors are applied to the definition.  It
2cccd0e3e9ea Numerous simplifications and removal of HOL-isms
paulson
parents: 3391
diff changeset
    66
* attempts to prove wellfoundedness of the given relation, simplifies the
2cccd0e3e9ea Numerous simplifications and removal of HOL-isms
paulson
parents: 3391
diff changeset
    67
* non-proved termination conditions, and finally attempts to prove the 
2cccd0e3e9ea Numerous simplifications and removal of HOL-isms
paulson
parents: 3391
diff changeset
    68
* simplified termination conditions.
2cccd0e3e9ea Numerous simplifications and removal of HOL-isms
paulson
parents: 3391
diff changeset
    69
*--------------------------------------------------------------------------*)
2cccd0e3e9ea Numerous simplifications and removal of HOL-isms
paulson
parents: 3391
diff changeset
    70
fun std_postprocessor ss =
2cccd0e3e9ea Numerous simplifications and removal of HOL-isms
paulson
parents: 3391
diff changeset
    71
  Prim.postprocess
4805
20d292c05e6c can prove the empty relation to be WF
paulson
parents: 4097
diff changeset
    72
   {WFtac      = REPEAT (ares_tac [wf_empty, wf_measure, wf_inv_image, 
20d292c05e6c can prove the empty relation to be WF
paulson
parents: 4097
diff changeset
    73
				   wf_lex_prod, wf_less_than, wf_trancl] 1),
3405
2cccd0e3e9ea Numerous simplifications and removal of HOL-isms
paulson
parents: 3391
diff changeset
    74
    terminator = asm_simp_tac ss 1
4097
ddd1c18121e0 CLASET';
wenzelm
parents: 3978
diff changeset
    75
		 THEN TRY(CLASET' (fn cs => best_tac
ddd1c18121e0 CLASET';
wenzelm
parents: 3978
diff changeset
    76
			  (cs addSDs [not0_implies_Suc] addss ss)) 1),
3405
2cccd0e3e9ea Numerous simplifications and removal of HOL-isms
paulson
parents: 3391
diff changeset
    77
    simplifier = Rules.simpl_conv ss []};
2112
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
    78
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
    79
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
    80
3391
5e45dd3b64e9 More de-HOLification: using Free, Const, etc. instead of mk_var, mk_const
paulson
parents: 3331
diff changeset
    81
val concl = #2 o Rules.dest_thm;
2112
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
    82
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
    83
(*---------------------------------------------------------------------------
3191
14bd6e5985f1 TFL now integrated with HOL (more work needed)
paulson
parents: 2467
diff changeset
    84
 * Defining a function with an associated termination relation. 
14bd6e5985f1 TFL now integrated with HOL (more work needed)
paulson
parents: 2467
diff changeset
    85
 *---------------------------------------------------------------------------*)
3331
c81c7f8ad333 Now checks the name of the function being defined
paulson
parents: 3302
diff changeset
    86
fun define_i thy fid R eqs = 
4970
8b65444edbb0 Changed require to requires for MLWorks
paulson
parents: 4856
diff changeset
    87
  let val dummy = Theory.requires thy "WF_Rel" "recursive function definitions"
3191
14bd6e5985f1 TFL now integrated with HOL (more work needed)
paulson
parents: 2467
diff changeset
    88
      val {functional,pats} = Prim.mk_functional thy eqs
3405
2cccd0e3e9ea Numerous simplifications and removal of HOL-isms
paulson
parents: 3391
diff changeset
    89
  in (Prim.wfrec_definition0 thy fid R functional, pats)
3191
14bd6e5985f1 TFL now integrated with HOL (more work needed)
paulson
parents: 2467
diff changeset
    90
  end;
14bd6e5985f1 TFL now integrated with HOL (more work needed)
paulson
parents: 2467
diff changeset
    91
14bd6e5985f1 TFL now integrated with HOL (more work needed)
paulson
parents: 2467
diff changeset
    92
(*lcp's version: takes strings; doesn't return "thm" 
3245
241838c01caf Removal of redundant code (unused or already present in Isabelle.
paulson
parents: 3208
diff changeset
    93
        (whose signature is a draft and therefore useless) *)
3331
c81c7f8ad333 Now checks the name of the function being defined
paulson
parents: 3302
diff changeset
    94
fun define thy fid R eqs = 
3191
14bd6e5985f1 TFL now integrated with HOL (more work needed)
paulson
parents: 2467
diff changeset
    95
  let fun read thy = readtm (sign_of thy) (TVar(("DUMMY",0),[])) 
3405
2cccd0e3e9ea Numerous simplifications and removal of HOL-isms
paulson
parents: 3391
diff changeset
    96
  in  define_i thy fid (read thy R) (map (read thy) eqs)  end
3191
14bd6e5985f1 TFL now integrated with HOL (more work needed)
paulson
parents: 2467
diff changeset
    97
  handle Utils.ERR {mesg,...} => error mesg;
14bd6e5985f1 TFL now integrated with HOL (more work needed)
paulson
parents: 2467
diff changeset
    98
14bd6e5985f1 TFL now integrated with HOL (more work needed)
paulson
parents: 2467
diff changeset
    99
(*---------------------------------------------------------------------------
14bd6e5985f1 TFL now integrated with HOL (more work needed)
paulson
parents: 2467
diff changeset
   100
 * Postprocess a definition made by "define". This is a separate stage of 
14bd6e5985f1 TFL now integrated with HOL (more work needed)
paulson
parents: 2467
diff changeset
   101
 * processing from the definition stage.
2112
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
   102
 *---------------------------------------------------------------------------*)
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
   103
local 
3391
5e45dd3b64e9 More de-HOLification: using Free, Const, etc. instead of mk_var, mk_const
paulson
parents: 3331
diff changeset
   104
structure R = Rules
2112
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
   105
structure U = Utils
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
   106
3191
14bd6e5985f1 TFL now integrated with HOL (more work needed)
paulson
parents: 2467
diff changeset
   107
(* The rest of these local definitions are for the tricky nested case *)
2112
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
   108
val solved = not o U.can S.dest_eq o #2 o S.strip_forall o concl
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
   109
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
   110
fun id_thm th = 
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
   111
   let val {lhs,rhs} = S.dest_eq(#2(S.strip_forall(#2 (R.dest_thm th))))
3391
5e45dd3b64e9 More de-HOLification: using Free, Const, etc. instead of mk_var, mk_const
paulson
parents: 3331
diff changeset
   112
   in lhs aconv rhs
2112
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
   113
   end handle _ => false
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
   114
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
   115
fun prover s = prove_goal HOL.thy s (fn _ => [fast_tac HOL_cs 1]);
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
   116
val P_imp_P_iff_True = prover "P --> (P= True)" RS mp;
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
   117
val P_imp_P_eq_True = P_imp_P_iff_True RS eq_reflection;
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
   118
fun mk_meta_eq r = case concl_of r of
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
   119
     Const("==",_)$_$_ => r
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
   120
  |   _$(Const("op =",_)$_$_) => r RS eq_reflection
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
   121
  |   _ => r RS P_imp_P_eq_True
3405
2cccd0e3e9ea Numerous simplifications and removal of HOL-isms
paulson
parents: 3391
diff changeset
   122
2cccd0e3e9ea Numerous simplifications and removal of HOL-isms
paulson
parents: 3391
diff changeset
   123
(*Is this the best way to invoke the simplifier??*)
3245
241838c01caf Removal of redundant code (unused or already present in Isabelle.
paulson
parents: 3208
diff changeset
   124
fun rewrite L = rewrite_rule (map mk_meta_eq (filter(not o id_thm) L))
2112
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
   125
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
   126
fun join_assums th = 
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
   127
  let val {sign,...} = rep_thm th
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
   128
      val tych = cterm_of sign
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
   129
      val {lhs,rhs} = S.dest_eq(#2 (S.strip_forall (concl th)))
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
   130
      val cntxtl = (#1 o S.strip_imp) lhs  (* cntxtl should = cntxtr *)
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
   131
      val cntxtr = (#1 o S.strip_imp) rhs  (* but union is solider *)
3245
241838c01caf Removal of redundant code (unused or already present in Isabelle.
paulson
parents: 3208
diff changeset
   132
      val cntxt = gen_union (op aconv) (cntxtl, cntxtr)
2112
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
   133
  in 
3191
14bd6e5985f1 TFL now integrated with HOL (more work needed)
paulson
parents: 2467
diff changeset
   134
    R.GEN_ALL 
14bd6e5985f1 TFL now integrated with HOL (more work needed)
paulson
parents: 2467
diff changeset
   135
      (R.DISCH_ALL 
14bd6e5985f1 TFL now integrated with HOL (more work needed)
paulson
parents: 2467
diff changeset
   136
         (rewrite (map (R.ASSUME o tych) cntxt) (R.SPEC_ALL th)))
2112
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
   137
  end
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
   138
  val gen_all = S.gen_all
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
   139
in
3405
2cccd0e3e9ea Numerous simplifications and removal of HOL-isms
paulson
parents: 3391
diff changeset
   140
fun proof_stage ss theory {f, R, rules, full_pats_TCs, TCs} =
3271
b873969b05d3 Basis library input/output primitives; currying the induction rule;
paulson
parents: 3245
diff changeset
   141
  let val dummy = prs "Proving induction theorem..  "
3191
14bd6e5985f1 TFL now integrated with HOL (more work needed)
paulson
parents: 2467
diff changeset
   142
      val ind = Prim.mk_induction theory f R full_pats_TCs
3405
2cccd0e3e9ea Numerous simplifications and removal of HOL-isms
paulson
parents: 3391
diff changeset
   143
      val dummy = prs "Proved induction theorem.\nPostprocessing..  "
2cccd0e3e9ea Numerous simplifications and removal of HOL-isms
paulson
parents: 3391
diff changeset
   144
      val {rules, induction, nested_tcs} = 
2cccd0e3e9ea Numerous simplifications and removal of HOL-isms
paulson
parents: 3391
diff changeset
   145
	  std_postprocessor ss theory {rules=rules, induction=ind, TCs=TCs}
3191
14bd6e5985f1 TFL now integrated with HOL (more work needed)
paulson
parents: 2467
diff changeset
   146
  in
14bd6e5985f1 TFL now integrated with HOL (more work needed)
paulson
parents: 2467
diff changeset
   147
  case nested_tcs
3271
b873969b05d3 Basis library input/output primitives; currying the induction rule;
paulson
parents: 3245
diff changeset
   148
  of [] => (writeln "Postprocessing done.";
3191
14bd6e5985f1 TFL now integrated with HOL (more work needed)
paulson
parents: 2467
diff changeset
   149
            {induction=induction, rules=rules,tcs=[]})
3271
b873969b05d3 Basis library input/output primitives; currying the induction rule;
paulson
parents: 3245
diff changeset
   150
  | L  => let val dummy = prs "Simplifying nested TCs..  "
2112
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
   151
              val (solved,simplified,stubborn) =
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
   152
               U.itlist (fn th => fn (So,Si,St) =>
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
   153
                     if (id_thm th) then (So, Si, th::St) else
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
   154
                     if (solved th) then (th::So, Si, St) 
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
   155
                     else (So, th::Si, St)) nested_tcs ([],[],[])
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
   156
              val simplified' = map join_assums simplified
3572
5ec1589eac1b Replaced clumsy rewriting by the new function simplify on thms.
nipkow
parents: 3556
diff changeset
   157
              val rewr = full_simplify (ss addsimps (solved @ simplified'));
3405
2cccd0e3e9ea Numerous simplifications and removal of HOL-isms
paulson
parents: 3391
diff changeset
   158
              val induction' = rewr induction
2cccd0e3e9ea Numerous simplifications and removal of HOL-isms
paulson
parents: 3391
diff changeset
   159
              and rules'     = rewr rules
3271
b873969b05d3 Basis library input/output primitives; currying the induction rule;
paulson
parents: 3245
diff changeset
   160
              val dummy = writeln "Postprocessing done."
2112
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
   161
          in
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
   162
          {induction = induction',
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
   163
               rules = rules',
3191
14bd6e5985f1 TFL now integrated with HOL (more work needed)
paulson
parents: 2467
diff changeset
   164
                 tcs = map (gen_all o S.rhs o #2 o S.strip_forall o concl)
14bd6e5985f1 TFL now integrated with HOL (more work needed)
paulson
parents: 2467
diff changeset
   165
                           (simplified@stubborn)}
2112
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
   166
          end
3391
5e45dd3b64e9 More de-HOLification: using Free, Const, etc. instead of mk_var, mk_const
paulson
parents: 3331
diff changeset
   167
  end;
3191
14bd6e5985f1 TFL now integrated with HOL (more work needed)
paulson
parents: 2467
diff changeset
   168
14bd6e5985f1 TFL now integrated with HOL (more work needed)
paulson
parents: 2467
diff changeset
   169
3302
404fe31fd8d2 New headers and other minor changes
paulson
parents: 3271
diff changeset
   170
(*lcp: curry the predicate of the induction rule*)
5103
866a281a8c2a Removed structure Prod_Syntax.
berghofe
parents: 4970
diff changeset
   171
fun curry_rule rl = split_rule_var
3271
b873969b05d3 Basis library input/output primitives; currying the induction rule;
paulson
parents: 3245
diff changeset
   172
                        (head_of (HOLogic.dest_Trueprop (concl_of rl)), 
b873969b05d3 Basis library input/output primitives; currying the induction rule;
paulson
parents: 3245
diff changeset
   173
			 rl);
b873969b05d3 Basis library input/output primitives; currying the induction rule;
paulson
parents: 3245
diff changeset
   174
3191
14bd6e5985f1 TFL now integrated with HOL (more work needed)
paulson
parents: 2467
diff changeset
   175
(*lcp: put a theorem into Isabelle form, using meta-level connectives*)
14bd6e5985f1 TFL now integrated with HOL (more work needed)
paulson
parents: 2467
diff changeset
   176
val meta_outer = 
3302
404fe31fd8d2 New headers and other minor changes
paulson
parents: 3271
diff changeset
   177
    curry_rule o standard o 
3271
b873969b05d3 Basis library input/output primitives; currying the induction rule;
paulson
parents: 3245
diff changeset
   178
    rule_by_tactic (REPEAT_FIRST (resolve_tac [allI, impI, conjI]
b873969b05d3 Basis library input/output primitives; currying the induction rule;
paulson
parents: 3245
diff changeset
   179
				  ORELSE' etac conjE));
3191
14bd6e5985f1 TFL now integrated with HOL (more work needed)
paulson
parents: 2467
diff changeset
   180
14bd6e5985f1 TFL now integrated with HOL (more work needed)
paulson
parents: 2467
diff changeset
   181
(*Strip off the outer !P*)
14bd6e5985f1 TFL now integrated with HOL (more work needed)
paulson
parents: 2467
diff changeset
   182
val spec'= read_instantiate [("x","P::?'b=>bool")] spec;
2112
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
   183
3405
2cccd0e3e9ea Numerous simplifications and removal of HOL-isms
paulson
parents: 3391
diff changeset
   184
val wf_rel_defs = [lex_prod_def, measure_def, inv_image_def];
2112
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
   185
3459
112cbb8301dc Removal of structure Context and its replacement by a theorem list of
paulson
parents: 3405
diff changeset
   186
(*Convert conclusion from = to ==*)
112cbb8301dc Removal of structure Context and its replacement by a theorem list of
paulson
parents: 3405
diff changeset
   187
val eq_reflect_list = map (fn th => (th RS eq_reflection) handle _ => th);
112cbb8301dc Removal of structure Context and its replacement by a theorem list of
paulson
parents: 3405
diff changeset
   188
112cbb8301dc Removal of structure Context and its replacement by a theorem list of
paulson
parents: 3405
diff changeset
   189
(*---------------------------------------------------------------------------
112cbb8301dc Removal of structure Context and its replacement by a theorem list of
paulson
parents: 3405
diff changeset
   190
 * Install the basic context notions. Others (for nat and list and prod) 
112cbb8301dc Removal of structure Context and its replacement by a theorem list of
paulson
parents: 3405
diff changeset
   191
 * have already been added in thry.sml
112cbb8301dc Removal of structure Context and its replacement by a theorem list of
paulson
parents: 3405
diff changeset
   192
 *---------------------------------------------------------------------------*)
112cbb8301dc Removal of structure Context and its replacement by a theorem list of
paulson
parents: 3405
diff changeset
   193
val defaultTflCongs = eq_reflect_list [Thms.LET_CONG, if_cong];
112cbb8301dc Removal of structure Context and its replacement by a theorem list of
paulson
parents: 3405
diff changeset
   194
112cbb8301dc Removal of structure Context and its replacement by a theorem list of
paulson
parents: 3405
diff changeset
   195
fun simplify_defn (ss, tflCongs) (thy,(id,pats)) =
3978
7e1cfed19d94 Sign.stamp_names_of;
wenzelm
parents: 3927
diff changeset
   196
   let val dummy = deny (id mem (Sign.stamp_names_of (sign_of thy)))
3208
8336393de482 Subst now moved to directory HOL
paulson
parents: 3191
diff changeset
   197
                        ("Recursive definition " ^ id ^ 
3245
241838c01caf Removal of redundant code (unused or already present in Isabelle.
paulson
parents: 3208
diff changeset
   198
                         " would clash with the theory of the same name!")
3405
2cccd0e3e9ea Numerous simplifications and removal of HOL-isms
paulson
parents: 3391
diff changeset
   199
       val def =  freezeT(get_def thy id)   RS   meta_eq_to_obj_eq
2cccd0e3e9ea Numerous simplifications and removal of HOL-isms
paulson
parents: 3391
diff changeset
   200
       val ss' = ss addsimps ((less_Suc_eq RS iffD2) :: wf_rel_defs)
3191
14bd6e5985f1 TFL now integrated with HOL (more work needed)
paulson
parents: 2467
diff changeset
   201
       val {theory,rules,TCs,full_pats_TCs,patterns} = 
3459
112cbb8301dc Removal of structure Context and its replacement by a theorem list of
paulson
parents: 3405
diff changeset
   202
                Prim.post_definition
112cbb8301dc Removal of structure Context and its replacement by a theorem list of
paulson
parents: 3405
diff changeset
   203
		   (ss', defaultTflCongs @ eq_reflect_list tflCongs)
112cbb8301dc Removal of structure Context and its replacement by a theorem list of
paulson
parents: 3405
diff changeset
   204
		   (thy, (def,pats))
3191
14bd6e5985f1 TFL now integrated with HOL (more work needed)
paulson
parents: 2467
diff changeset
   205
       val {lhs=f,rhs} = S.dest_eq(concl def)
14bd6e5985f1 TFL now integrated with HOL (more work needed)
paulson
parents: 2467
diff changeset
   206
       val (_,[R,_]) = S.strip_comb rhs
14bd6e5985f1 TFL now integrated with HOL (more work needed)
paulson
parents: 2467
diff changeset
   207
       val {induction, rules, tcs} = 
3405
2cccd0e3e9ea Numerous simplifications and removal of HOL-isms
paulson
parents: 3391
diff changeset
   208
             proof_stage ss' theory 
3245
241838c01caf Removal of redundant code (unused or already present in Isabelle.
paulson
parents: 3208
diff changeset
   209
               {f = f, R = R, rules = rules,
241838c01caf Removal of redundant code (unused or already present in Isabelle.
paulson
parents: 3208
diff changeset
   210
                full_pats_TCs = full_pats_TCs,
241838c01caf Removal of redundant code (unused or already present in Isabelle.
paulson
parents: 3208
diff changeset
   211
                TCs = TCs}
3191
14bd6e5985f1 TFL now integrated with HOL (more work needed)
paulson
parents: 2467
diff changeset
   212
       val rules' = map (standard o normalize_thm [RSmp]) (R.CONJUNCTS rules)
14bd6e5985f1 TFL now integrated with HOL (more work needed)
paulson
parents: 2467
diff changeset
   213
   in  {induct = meta_outer
3245
241838c01caf Removal of redundant code (unused or already present in Isabelle.
paulson
parents: 3208
diff changeset
   214
                  (normalize_thm [RSspec,RSmp] (induction RS spec')), 
241838c01caf Removal of redundant code (unused or already present in Isabelle.
paulson
parents: 3208
diff changeset
   215
        rules = rules', 
241838c01caf Removal of redundant code (unused or already present in Isabelle.
paulson
parents: 3208
diff changeset
   216
        tcs = (termination_goals rules') @ tcs}
3191
14bd6e5985f1 TFL now integrated with HOL (more work needed)
paulson
parents: 2467
diff changeset
   217
   end
3391
5e45dd3b64e9 More de-HOLification: using Free, Const, etc. instead of mk_var, mk_const
paulson
parents: 3331
diff changeset
   218
  handle Utils.ERR {mesg,func,module} => 
5e45dd3b64e9 More de-HOLification: using Free, Const, etc. instead of mk_var, mk_const
paulson
parents: 3331
diff changeset
   219
               error (mesg ^ 
3405
2cccd0e3e9ea Numerous simplifications and removal of HOL-isms
paulson
parents: 3391
diff changeset
   220
		      "\n    (In TFL function " ^ module ^ "." ^ func ^ ")");
2112
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
   221
end;
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
   222
3191
14bd6e5985f1 TFL now integrated with HOL (more work needed)
paulson
parents: 2467
diff changeset
   223
(*---------------------------------------------------------------------------
14bd6e5985f1 TFL now integrated with HOL (more work needed)
paulson
parents: 2467
diff changeset
   224
 *
14bd6e5985f1 TFL now integrated with HOL (more work needed)
paulson
parents: 2467
diff changeset
   225
 *     Definitions with synthesized termination relation temporarily
14bd6e5985f1 TFL now integrated with HOL (more work needed)
paulson
parents: 2467
diff changeset
   226
 *     deleted -- it's not clear how to integrate this facility with
14bd6e5985f1 TFL now integrated with HOL (more work needed)
paulson
parents: 2467
diff changeset
   227
 *     the Isabelle theory file scheme, which restricts
14bd6e5985f1 TFL now integrated with HOL (more work needed)
paulson
parents: 2467
diff changeset
   228
 *     inference at theory-construction time.
14bd6e5985f1 TFL now integrated with HOL (more work needed)
paulson
parents: 2467
diff changeset
   229
 *
2112
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
   230
3391
5e45dd3b64e9 More de-HOLification: using Free, Const, etc. instead of mk_var, mk_const
paulson
parents: 3331
diff changeset
   231
local structure R = Rules
2112
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
   232
in
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
   233
fun function theory eqs = 
3208
8336393de482 Subst now moved to directory HOL
paulson
parents: 3191
diff changeset
   234
 let val dummy = prs "Making definition..   "
2112
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
   235
     val {rules,R,theory,full_pats_TCs,...} = Prim.lazyR_def theory eqs
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
   236
     val f = func_of_cond_eqn (concl(R.CONJUNCT1 rules handle _ => rules))
3208
8336393de482 Subst now moved to directory HOL
paulson
parents: 3191
diff changeset
   237
     val dummy = prs "Definition made.\n"
8336393de482 Subst now moved to directory HOL
paulson
parents: 3191
diff changeset
   238
     val dummy = prs "Proving induction theorem..  "
2112
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
   239
     val induction = Prim.mk_induction theory f R full_pats_TCs
3208
8336393de482 Subst now moved to directory HOL
paulson
parents: 3191
diff changeset
   240
     val dummy = prs "Induction theorem proved.\n"
2112
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
   241
 in {theory = theory, 
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
   242
     eq_ind = standard (induction RS (rules RS conjI))}
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
   243
 end
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
   244
end;
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
   245
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
   246
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
   247
fun lazyR_def theory eqs = 
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
   248
   let val {rules,theory, ...} = Prim.lazyR_def theory eqs
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
   249
   in {eqns=rules, theory=theory}
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
   250
   end
3391
5e45dd3b64e9 More de-HOLification: using Free, Const, etc. instead of mk_var, mk_const
paulson
parents: 3331
diff changeset
   251
   handle    e              => print_exn e;
3191
14bd6e5985f1 TFL now integrated with HOL (more work needed)
paulson
parents: 2467
diff changeset
   252
 *
14bd6e5985f1 TFL now integrated with HOL (more work needed)
paulson
parents: 2467
diff changeset
   253
 *
14bd6e5985f1 TFL now integrated with HOL (more work needed)
paulson
parents: 2467
diff changeset
   254
 *---------------------------------------------------------------------------*)
2112
3902e9af752f Konrad Slind's TFL
paulson
parents:
diff changeset
   255
end;