Skip to content

Commit

Permalink
Add (HasType (Tm_type u) (Tm_type (U_succ u)))
Browse files Browse the repository at this point in the history
  • Loading branch information
nikswamy committed Jan 13, 2025
1 parent e0d07a2 commit 9fee831
Showing 1 changed file with 6 additions and 0 deletions.
6 changes: 6 additions & 0 deletions src/smtencoding/FStarC.SMTEncoding.Term.fst
Original file line number Diff line number Diff line change
Expand Up @@ -1064,6 +1064,11 @@ and mkPrelude z3options =
:pattern ((Valid t))\n\
:qid __prelude_valid_elim)))\n"
in
let tm_type_typing =
"(assert (forall ((u Universe) (t Term))\n\
(! (iff (HasType (Tm_type u) t)\n\
(= t (Tm_type (U_succ u))))\n\
:pattern ((HasType (Tm_type u) t)))))\n" in
basic
^ bcons
^ precedes_partial_app
Expand All @@ -1074,6 +1079,7 @@ and mkPrelude z3options =
^ (if FStarC.Options.smtencoding_valid_elim()
then valid_elim
else "")
^ tm_type_typing
let declsToSmt z3options decls = List.map (declToSmt z3options) decls |> String.concat "\n"
let declToSmt_no_caps z3options decl = declToSmt' false z3options decl
Expand Down

0 comments on commit 9fee831

Please sign in to comment.