Skip to content

Commit

Permalink
evarsolve transp_state and comments fixes
Browse files Browse the repository at this point in the history
  • Loading branch information
mattam82 committed Feb 8, 2019
1 parent b74aaa4 commit ab63977
Show file tree
Hide file tree
Showing 2 changed files with 8 additions and 8 deletions.
10 changes: 5 additions & 5 deletions pretyping/evarsolve.ml
Original file line number Diff line number Diff line change
Expand Up @@ -26,9 +26,9 @@ open Pretype_errors

type unify_flags = {
modulo_betaiota: bool;
open_ts : transparent_state;
closed_ts : transparent_state;
subterm_ts : transparent_state;
open_ts : TransparentState.t;
closed_ts : TransparentState.t;
subterm_ts : TransparentState.t;
frozen_evars : Evar.Set.t;
allow_K_at_toplevel : bool;
with_cs : bool }
Expand Down Expand Up @@ -1442,8 +1442,8 @@ let occur_evar_upto_types sigma n c =
try occur_rec c; false with Occur -> true

let instantiate_evar unify flags evd evk body =
(** Check instance freezing the evar to be defined, as
checking could involve the same evar definition problem again otherwise *)
(* Check instance freezing the evar to be defined, as
checking could involve the same evar definition problem again otherwise *)
let flags = { flags with frozen_evars = Evar.Set.add evk flags.frozen_evars } in
let evd' = check_evar_instance unify flags evd evk body in
Evd.define evk body evd'
Expand Down
6 changes: 3 additions & 3 deletions pretyping/evarsolve.mli
Original file line number Diff line number Diff line change
Expand Up @@ -19,11 +19,11 @@ val of_alias : alias -> EConstr.t
type unify_flags = {
modulo_betaiota : bool;
(* Enable beta-iota reductions during unification *)
open_ts : Names.transparent_state;
open_ts : TransparentState.t;
(* Enable delta reduction according to open_ts for open terms *)
closed_ts : Names.transparent_state;
closed_ts : TransparentState.t;
(* Enable delta reduction according to closed_ts for closed terms (when calling conversion) *)
subterm_ts : Names.transparent_state;
subterm_ts : TransparentState.t;
(* Enable delta reduction according to subterm_ts for selection of subterms during higher-order
unifications. *)
frozen_evars : Evar.Set.t;
Expand Down

0 comments on commit ab63977

Please sign in to comment.