aboutsummaryrefslogtreecommitdiffhomepage
path: root/proofs/refiner.ml
diff options
context:
space:
mode:
authorGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2014-04-06 19:08:11 +0200
committerGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2014-04-06 19:18:11 +0200
commitaba9691ef2d8d6ffd184e3d97de47d9c48f1a1b3 (patch)
tree1dfc529b52c8a46d80bf82305b4b20c908a64c6b /proofs/refiner.ml
parentb3b302837a5a9ff4e50a7f69ecb3fb333c94bf01 (diff)
Removing unused functions in Refiner.
Diffstat (limited to 'proofs/refiner.ml')
-rw-r--r--proofs/refiner.ml43
1 files changed, 0 insertions, 43 deletions
diff --git a/proofs/refiner.ml b/proofs/refiner.ml
index 7e80b40e5..9a78a79fd 100644
--- a/proofs/refiner.ml
+++ b/proofs/refiner.ml
@@ -315,49 +315,6 @@ let rec tclREPEAT_MAIN t g =
(tclORELSE (tclTHEN_i t (fun i -> if Int.equal i 1 then (tclREPEAT_MAIN t) else
tclIDTAC)) tclIDTAC) g
-(*s Tactics handling a list of goals. *)
-
-type tactic_list = (goal list sigma) -> (goal list sigma)
-
-(* Functions working on goal list for correct backtracking in Prolog *)
-
-let tclFIRSTLIST = tclFIRST
-let tclIDTAC_list gls = gls
-
-(* first_goal : goal list sigma -> goal sigma *)
-
-let first_goal gls =
- let gl = gls.it and sig_0 = gls.sigma in
- if List.is_empty gl then error "first_goal";
- { it = List.hd gl; sigma = sig_0; }
-
-(* goal_goal_list : goal sigma -> goal list sigma *)
-
-let goal_goal_list gls =
- let gl = gls.it and sig_0 = gls.sigma in
- { it = [gl]; sigma = sig_0; }
-
-(* tactic -> tactic_list : Apply a tactic to the first goal in the list *)
-
-let apply_tac_list tac glls =
- let (sigr,lg) = unpackage glls in
- match lg with
- | (g1::rest) ->
- let gl = apply_sig_tac sigr tac g1 in
- repackage sigr (gl@rest)
- | _ -> error "apply_tac_list"
-
-let then_tactic_list tacl1 tacl2 glls =
- let glls1 = tacl1 glls in
- let glls2 = tacl2 glls1 in
- glls2
-
-(* Transform a tactic_list into a tactic *)
-
-let tactic_list_tactic tac gls =
- let glres = tac (goal_goal_list gls) in
- glres
-
(* Change evars *)
let tclEVARS sigma gls = tclIDTAC {gls with sigma=sigma}