Skip to content

Commit

Permalink
Merge pull request #3413 from mtzguido/imp_refactor
Browse files Browse the repository at this point in the history
Refactoring implicit instantiation
  • Loading branch information
mtzguido authored Aug 26, 2024
2 parents 04413e8 + 0ab882f commit a26252e
Show file tree
Hide file tree
Showing 10 changed files with 304 additions and 392 deletions.
4 changes: 4 additions & 0 deletions ocaml/fstar-lib/generated/FStar_Syntax_Subst.ml

Some generated files are not rendered by default. Learn more about how customized files appear on GitHub.

249 changes: 65 additions & 184 deletions ocaml/fstar-lib/generated/FStar_TypeChecker_TcTerm.ml

Large diffs are not rendered by default.

243 changes: 149 additions & 94 deletions ocaml/fstar-lib/generated/FStar_TypeChecker_Util.ml

Some generated files are not rendered by default. Learn more about how customized files appear on GitHub.

1 change: 1 addition & 0 deletions src/syntax/FStar.Syntax.Subst.fst
Original file line number Diff line number Diff line change
Expand Up @@ -294,6 +294,7 @@ let subst_binder' s b =
b.binder_positivity
(b.binder_attrs |> List.map (subst' s))

let subst_binder s (b:binder) = subst_binder' ([s], NoUseRange) b

let subst_binders' s bs =
bs |> List.mapi (fun i b ->
Expand Down
1 change: 1 addition & 0 deletions src/syntax/FStar.Syntax.Subst.fsti
Original file line number Diff line number Diff line change
Expand Up @@ -31,6 +31,7 @@ val subst_aqual: list subst_elt -> aqual -> aqual
val subst_ascription: list subst_elt -> ascription -> ascription
val subst_decreasing_order:
list subst_elt -> decreases_order -> decreases_order
val subst_binder: list subst_elt -> binder -> binder
val subst_binders: list subst_elt -> binders -> binders
val subst_residual_comp:list subst_elt -> residual_comp -> residual_comp
val compress: term -> term
Expand Down
Loading

0 comments on commit a26252e

Please sign in to comment.