Skip to content

Commit

Permalink
Stop doing early universe minimization and nf_evar in abstract
Browse files Browse the repository at this point in the history
  • Loading branch information
SkySkimmer committed Sep 27, 2023
1 parent 3a95cfb commit fea5fcc
Showing 1 changed file with 0 additions and 6 deletions.
6 changes: 0 additions & 6 deletions vernac/declare.ml
Original file line number Diff line number Diff line change
Expand Up @@ -1900,12 +1900,6 @@ let build_by_tactic env ~uctx ~poly ~typ tac =
cb, ce.proof_entry_type, ce.proof_entry_universes, status, uctx

let declare_abstract ~name ~poly ~kind ~sign ~secsign ~opaque ~solve_tac sigma concl =
let sigma, concl =
(* FIXME: should be done only if the tactic succeeds *)
(* XXX maybe we can fix now that we support evars *)
let sigma = Evd.minimize_universes sigma in
sigma, Evarutil.nf_evar sigma concl
in
let (const, safe, sigma') =
try build_constant_by_tactic ~warn_incomplete:false ~name ~opaque:Vernacexpr.Transparent ~poly ~sigma ~sign:secsign concl solve_tac
with Logic_monad.TacticFailure e as src ->
Expand Down

0 comments on commit fea5fcc

Please sign in to comment.