aboutsummaryrefslogtreecommitdiffhomepage
path: root/proofs/proof_trees.ml
diff options
context:
space:
mode:
Diffstat (limited to 'proofs/proof_trees.ml')
-rw-r--r--proofs/proof_trees.ml19
1 files changed, 0 insertions, 19 deletions
diff --git a/proofs/proof_trees.ml b/proofs/proof_trees.ml
index 967b3edaf..445e19967 100644
--- a/proofs/proof_trees.ml
+++ b/proofs/proof_trees.ml
@@ -70,25 +70,6 @@ let is_tactic_proof pf = match pf.ref with
(* Constraints for existential variables *)
(*******************************************************************)
-(* A readable constraint is a global constraint plus a focus set
- of existential variables and a signature. *)
-
-(* Functions on readable constraints *)
-
-let mt_evcty gc =
- { it = empty_named_context; sigma = gc }
-
-let rc_of_gc evds gl =
- { it = gl.evar_hyps; sigma = evds }
-
-let rc_add evc (k,v) =
- { it = evc.it;
- sigma = Evd.add evc.sigma k v }
-
-let get_hyps evc = evc.it
-let get_env evc = Global.env_of_context evc.it
-let get_gc evc = evc.sigma
-
let pf_lookup_name_as_renamed env ccl s =
Detyping.lookup_name_as_renamed env ccl s