aboutsummaryrefslogtreecommitdiffhomepage
path: root/plugins/cc
diff options
context:
space:
mode:
authorGravatar Gaetan Gilbert <gaetan.gilbert@ens-lyon.fr>2017-04-27 21:58:52 +0200
committerGravatar Gaetan Gilbert <gaetan.gilbert@ens-lyon.fr>2017-04-27 21:58:52 +0200
commit9a48211ea8439a8502145e508b70ede9b5929b2f (patch)
tree55b533fdf2e2237e675dfddccad9f3bb1d8cc23c /plugins/cc
parenta77734ad64fff2396b161308099923037fb5d8a1 (diff)
Post-rebase warnings (unused opens and 2 unused values)
Diffstat (limited to 'plugins/cc')
-rw-r--r--plugins/cc/cctac.ml2
-rw-r--r--plugins/cc/cctac.mli1
2 files changed, 0 insertions, 3 deletions
diff --git a/plugins/cc/cctac.ml b/plugins/cc/cctac.ml
index 00b31ccce..7c5efaea3 100644
--- a/plugins/cc/cctac.ml
+++ b/plugins/cc/cctac.ml
@@ -15,13 +15,11 @@ open Declarations
open Term
open EConstr
open Vars
-open Tacmach
open Tactics
open Typing
open Ccalgo
open Ccproof
open Pp
-open CErrors
open Util
open Proofview.Notations
diff --git a/plugins/cc/cctac.mli b/plugins/cc/cctac.mli
index 5099d847b..b4bb62be8 100644
--- a/plugins/cc/cctac.mli
+++ b/plugins/cc/cctac.mli
@@ -8,7 +8,6 @@
(************************************************************************)
open EConstr
-open Proof_type
val proof_tac: Ccproof.proof -> unit Proofview.tactic