Skip to content

Commit

Permalink
Merge pull request #1176 from FStarLang/tchajed_inline_types
Browse files Browse the repository at this point in the history
Inline definitions while computing ML types
  • Loading branch information
msprotz authored Aug 7, 2017
2 parents 4f7e25b + 879fc34 commit 5269ce2
Showing 1 changed file with 2 additions and 2 deletions.
4 changes: 2 additions & 2 deletions src/extraction/FStar.Extraction.ML.Term.fs
Original file line number Diff line number Diff line change
Expand Up @@ -433,11 +433,11 @@ let rec term_as_mlty (g:env) (t0:term) : mlty =
end
| _ -> false
in
let t = N.normalize [N.Beta; N.Eager_unfolding; N.Iota; N.Zeta; N.EraseUniverses; N.AllowUnboundUniverses] g.tcenv t0 in
let t = N.normalize [N.Beta; N.Eager_unfolding; N.Iota; N.Zeta; N.Inlining; N.EraseUniverses; N.AllowUnboundUniverses] g.tcenv t0 in
let mlt = term_as_mlty' g t in
if is_top_ty mlt
then //Try normalizing t fully, this time with Delta steps, and translate again, to see if we can get a better translation for it
let t = N.normalize [N.Beta; N.Eager_unfolding; N.UnfoldUntil Delta_constant; N.Iota; N.Zeta; N.EraseUniverses; N.AllowUnboundUniverses] g.tcenv t0 in
let t = N.normalize [N.Beta; N.Eager_unfolding; N.UnfoldUntil Delta_constant; N.Iota; N.Zeta; N.Inlining; N.EraseUniverses; N.AllowUnboundUniverses] g.tcenv t0 in
term_as_mlty' g t
else mlt

Expand Down

0 comments on commit 5269ce2

Please sign in to comment.