aboutsummaryrefslogtreecommitdiff
path: root/proofs/proofview.ml
diff options
context:
space:
mode:
authorArnaud Spiwack2014-10-17 16:25:03 +0200
committerArnaud Spiwack2014-10-22 07:31:45 +0200
commitf613bad27923c0154d5576e87a9dc104f024eb8d (patch)
treeb2cff1b2cd67342eb3468295d598fa68cbddc521 /proofs/proofview.ml
parentaa64260119704620540017a23815cd7c40c3cff3 (diff)
Proofview: clean up commented out code.
Diffstat (limited to 'proofs/proofview.ml')
-rw-r--r--proofs/proofview.ml6
1 files changed, 0 insertions, 6 deletions
diff --git a/proofs/proofview.ml b/proofs/proofview.ml
index 98a6e7c140..836101ce54 100644
--- a/proofs/proofview.ml
+++ b/proofs/proofview.ml
@@ -156,12 +156,6 @@ let return_constr { solution = defs } c = Evarutil.nf_evar defs c
let partial_proof entry pv = List.map (return_constr pv) (List.map fst entry)
-(* let return { initial=init; solution=defs } = *)
-(* let evdref = ref defs in *)
-(* let nf,subst = Evarutil.e_nf_evars_and_universes evdref in *)
-(* ((List.map (fun (c,t) -> (nf c, nf t)) init, subst), *)
-(* Evd.universe_context !evdref) *)
-
(* spiwack: this function should probably go in the Util section,
but I'd rather have Util (or a separate module for lists)
raise proper exceptions before *)