aboutsummaryrefslogtreecommitdiffhomepage
path: root/contrib/first-order/rules.ml
blob: be91c9ec5d1e849c796217e05f55a58c62bde850 (plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
16
17
18
19
20
21
22
23
24
25
26
27
28
29
30
31
32
33
34
35
36
37
38
39
40
41
42
43
44
45
46
47
48
49
50
51
52
53
54
55
56
57
58
59
60
61
62
63
64
65
66
67
68
69
70
71
72
73
74
75
76
77
78
79
80
81
82
83
84
85
86
87
88
89
90
91
92
93
94
95
96
97
98
99
100
101
102
103
104
105
106
107
108
109
110
111
112
113
114
115
116
117
118
119
120
121
122
123
124
125
126
127
128
129
130
131
132
133
134
135
136
137
138
139
140
141
142
143
144
145
146
147
148
149
150
151
152
153
154
155
156
157
158
159
160
161
162
163
164
165
166
167
168
169
170
171
172
173
174
175
176
177
178
179
180
181
182
183
184
185
186
187
188
189
190
191
192
(***********************************************************************)
(*  v      *   The Coq Proof Assistant  /  The Coq Development Team    *)
(* <O___,, *        INRIA-Rocquencourt  &  LRI-CNRS-Orsay              *)
(*   \VV/  *************************************************************)
(*    //   *      This file is distributed under the terms of the      *)
(*         *       GNU Lesser General Public License Version 2.1       *)
(***********************************************************************)

(* $Id$ *)

open Util
open Names
open Term
open Tacmach
open Tactics
open Tacticals
open Termops
open Declarations
open Formula
open Sequent
open Libnames

type seqtac= (Sequent.t -> tactic) -> Sequent.t -> tactic

type lseqtac= global_reference -> seqtac

let wrap n b tacrec seq gls=
  check_for_interrupt ();
  let nc=pf_hyps gls in
  let env=pf_env gls in
  let rec aux i nc ctx=
    if i<=0 then seq else 
      match nc with
	  []->anomaly "Not the expected number of hyps"
	| ((id,_,typ) as nd)::q->  
	    if occur_var env id (pf_concl gls) || 
	      List.exists (occur_var_in_decl env id) ctx then
		(aux (i-1) q (nd::ctx))
	    else
	      add_formula false (VarRef id) typ (aux (i-1) q (nd::ctx)) gls in
  let seq1=aux n nc [] in
  let seq2=if b then 
    add_formula true dummy_id (pf_concl gls) seq1 gls else seq1 in
    tacrec seq2 gls

let id_of_global=function
    VarRef id->id
  | _->assert false

let clear_global=function
    VarRef id->clear [id]
  | _->tclIDTAC
      

(* connection rules *)

let axiom_tac t seq=
  try exact_no_check (constr_of_reference (find_left t seq)) 
  with Not_found->tclFAIL 0 "No axiom link" 

let ll_atom_tac a id tacrec seq=
  try 
    tclTHENLIST
      [generalize [mkApp(constr_of_reference id,
			 [|constr_of_reference (find_left a seq)|])];
       clear_global id;
       introf;
       wrap 1 false tacrec seq] 
  with Not_found->tclFAIL 0 "No link" 

(* right connectives rules *)

let and_tac tacrec seq=
  tclTHEN simplest_split (wrap 0 true tacrec seq)

let or_tac tacrec seq=
  any_constructor (Some (tclSOLVE [wrap 0 true tacrec seq]))

let arrow_tac tacrec seq=
  tclTHEN introf (wrap 1 true tacrec seq)
   
(* left connectives rules *)

let left_and_tac ind id tacrec seq=
  let n=(construct_nhyps ind).(0) in  
    tclTHENLIST 
      [simplest_elim (constr_of_reference id);
       clear_global id; 
       tclDO n introf;
       wrap n false tacrec seq]

let left_or_tac ind id tacrec seq=
  let v=construct_nhyps ind in  
  let f n=
    tclTHENLIST
      [clear_global id;
       tclDO n introf;
       wrap n false tacrec seq] in
    tclTHENSV
      (simplest_elim (constr_of_reference id))
      (Array.map f v)

let left_false_tac id=
  simplest_elim (constr_of_reference id)

(* left arrow connective rules *)

(* We use this function for false, and, or, exists *)

let ll_ind_tac ind largs id tacrec seq gl= 
  (try
     let rcs=ind_hyps 0 ind largs in
     let vargs=Array.of_list largs in
	     (* construire le terme  H->B, le generaliser etc *)   
     let myterm i=
       let rc=rcs.(i) in
       let p=List.length rc in
       let cstr=mkApp ((mkConstruct (ind,(i+1))),vargs) in
       let vars=Array.init p (fun j->mkRel (p-j)) in
       let capply=mkApp ((lift p cstr),vars) in
       let head=mkApp ((lift p (constr_of_reference id)),[|capply|]) in
	 Sign.it_mkLambda_or_LetIn head rc in
       let lp=Array.length rcs in
       let newhyps=list_tabulate myterm lp in
	 tclTHENLIST 
	   [generalize newhyps;
	    clear_global id;
	    tclDO lp introf;
	    wrap lp false tacrec seq]
   with Invalid_argument _ ->tclFAIL 0 "") gl

let ll_arrow_tac a b c id tacrec seq=
  let cc=mkProd(Anonymous,a,(lift 1 b)) in
  let d=mkLambda (Anonymous,b,
		  mkApp ((constr_of_reference id),
			 [|mkLambda (Anonymous,(lift 1 a),(mkRel 2))|])) in
    tclTHENS (cut c)
      [tclTHENLIST
	 [introf;
	  clear_global id;
	  wrap 1 false tacrec seq];
       tclTHENS (cut cc) 
         [exact_no_check (constr_of_reference id); 
	  tclTHENLIST 
	    [generalize [d];
	     introf;
	     clear_global id;
	     tclSOLVE [wrap 1 true tacrec seq]]]]

(* quantifier rules (easy side) *)

let forall_tac tacrec seq=
  tclTHEN introf (wrap 0 true tacrec seq)

let left_exists_tac ind id tacrec seq=
  let n=(construct_nhyps ind).(0) in  
    tclTHENLIST
      [simplest_elim (constr_of_reference id);
       clear_global id;
       tclDO n introf;
       (wrap (n-1) false tacrec seq)]

let ll_forall_tac prod id tacrec seq=
  tclTHENS (cut prod)
    [tclTHENLIST
       [introf;
	(fun gls->
	   let id0=pf_nth_hyp_id gls 1 in
	   let term=mkApp((constr_of_reference id),[|mkVar(id0)|]) in
	     tclTHEN (generalize [term]) (clear [id0]) gls);  
	clear_global id;
	introf;
	tclSOLVE [wrap 1 false tacrec (deepen seq)]];
     tclSOLVE [wrap 0 true tacrec (deepen seq)]]

(* rules for instantiation with unification moved to instances.ml *)

(* special for compatibility with old Intuition *)

let constant str = Coqlib.gen_constant "User" ["Init";"Logic"] str

let defined_connectives=lazy
  [[],EvalConstRef (destConst (constant "not"));
   [],EvalConstRef (destConst (constant "iff"))]

let normalize_evaluables=
  onAllClauses
    (function 
	 None->unfold_in_concl (Lazy.force defined_connectives)
       | Some id-> 
	   unfold_in_hyp (Lazy.force defined_connectives) 
	   (Tacexpr.InHypType id))