aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
-rw-r--r--tactics/setoid_replace.ml2
-rw-r--r--tactics/tacinterp.ml3
-rw-r--r--tactics/tacticals.ml1
-rw-r--r--tactics/tactics.ml8
4 files changed, 6 insertions, 8 deletions
diff --git a/tactics/setoid_replace.ml b/tactics/setoid_replace.ml
index e44b66bd4..3efd23f6a 100644
--- a/tactics/setoid_replace.ml
+++ b/tactics/setoid_replace.ml
@@ -53,7 +53,7 @@ let global_constant dir s =Coqlib.gen_constant "Setoid_replace" ("Init"::dir) s
let current_constant id =
try
- Declare.global_reference id
+ global_reference id
with Not_found ->
anomaly ("Setoid: cannot find "^(string_of_id id))
diff --git a/tactics/tacinterp.ml b/tactics/tacinterp.ml
index e7f4fff8b..536ddfb66 100644
--- a/tactics/tacinterp.ml
+++ b/tactics/tacinterp.ml
@@ -35,7 +35,6 @@ open Topconstr
open Ast
open Term
open Termops
-open Declare
open Tacexpr
open Safe_typing
open Typing
@@ -122,7 +121,7 @@ let make_hyps = List.map (fun (id,_,typ) -> (id, typ))
(* Transforms an id into a constr if possible, or fails *)
let constr_of_id env id =
- construct_reference (Some (Environ.named_context env)) id
+ construct_reference (Environ.named_context env) id
(* To embed several objects in Coqast.t *)
let ((tactic_in : (interp_sign -> raw_tactic_expr) -> Dyn.t),
diff --git a/tactics/tacticals.ml b/tactics/tacticals.ml
index 475b29be4..b5fc4e253 100644
--- a/tactics/tacticals.ml
+++ b/tactics/tacticals.ml
@@ -19,7 +19,6 @@ open Inductive
open Reduction
open Environ
open Libnames
-open Declare
open Refiner
open Tacmach
open Clenv
diff --git a/tactics/tactics.ml b/tactics/tactics.ml
index 1b9f86023..41dce0fef 100644
--- a/tactics/tactics.ml
+++ b/tactics/tactics.ml
@@ -21,7 +21,6 @@ open Inductiveops
open Reductionops
open Environ
open Libnames
-open Declare
open Evd
open Pfedit
open Tacred
@@ -229,12 +228,13 @@ let unfold_constr = function
(*******************************************)
let is_section_variable id =
- try let _ = Declare.find_section_variable id in true with Not_found -> false
+ try let _ = Sign.lookup_named id (Global.named_context()) in true
+ with Not_found -> false
let next_global_ident_from id avoid =
let rec next_rec id =
let id = next_ident_away_from id avoid in
- if is_section_variable id || not (Declare.is_global id) then
+ if is_section_variable id || not (is_global id) then
id
else
next_rec (lift_ident id)
@@ -243,7 +243,7 @@ let next_global_ident_from id avoid =
let next_global_ident_away id avoid =
let id = next_ident_away id avoid in
- if is_section_variable id || not (Declare.is_global id) then
+ if is_section_variable id || not (is_global id) then
id
else
next_global_ident_from (lift_ident id) avoid