From 23f4804b50307766219392229757e75da9aa41d9 Mon Sep 17 00:00:00 2001 From: Matthieu Sozeau Date: Wed, 18 Jun 2014 17:16:59 +0200 Subject: Proofs now take and return an evar_universe_context, simplifying interfaces and avoiding explicit substitutions and merging of contexts, e.g. in obligations.ml. The context produced by typechecking a statement is passed in the proof, allowing the universe name context to be correctly folded as well. Mainly an API cleanup. --- tactics/tacinterp.ml | 3 +-- 1 file changed, 1 insertion(+), 2 deletions(-) (limited to 'tactics/tacinterp.ml') diff --git a/tactics/tacinterp.ml b/tactics/tacinterp.ml index 1d76f4afd..aafe6f2f7 100644 --- a/tactics/tacinterp.ml +++ b/tactics/tacinterp.ml @@ -2060,8 +2060,7 @@ let _ = if has_type arg (glbwit wit_tactic) then let tac = out_gen (glbwit wit_tactic) arg in let tac = interp_tactic ist tac in - let ctx = Evd.universe_context_set sigma in - let prf = Proof.start sigma [env, (ty, ctx)] in + let prf = Proof.start sigma [env, ty] in let (prf, _) = try Proof.run_tactic env tac prf with Proof_errors.TacticFailure e as src -> -- cgit v1.2.3