Skip to content

Commit

Permalink
Merge pull request #3556 from mtzguido/move
Browse files Browse the repository at this point in the history
ulib: move a type into stubs
  • Loading branch information
mtzguido authored Oct 10, 2024
2 parents 59f13d3 + 724725e commit 9ec5695
Show file tree
Hide file tree
Showing 6 changed files with 16 additions and 16 deletions.
2 changes: 1 addition & 1 deletion ocaml/fstar-lib/generated/FStar_Reflection_TermEq.ml

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

9 changes: 4 additions & 5 deletions ocaml/fstar-lib/generated/FStar_Reflection_Typing.ml

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

5 changes: 2 additions & 3 deletions ocaml/fstar-lib/generated/FStar_Tactics_NamedView.ml

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

7 changes: 0 additions & 7 deletions ulib/FStar.Stubs.Reflection.Types.fsti
Original file line number Diff line number Diff line change
Expand Up @@ -40,11 +40,4 @@ type univ_name = ident
type typ = term
type binders = list binder

(*
* match e as binder returns t|C
*
* the bool says whether returns (bool = false) or returns$ (bool = true, use type equality
*)
type match_returns_ascription = binder & (either term comp & option term & bool)

type decls = list sigelt
1 change: 1 addition & 0 deletions ulib/FStar.Stubs.Reflection.V1.Data.fsti
Original file line number Diff line number Diff line change
Expand Up @@ -22,6 +22,7 @@ open FStar.Stubs.Reflection.V2.Data {}
open FStar.Stubs.Reflection.V2.Builtins {}

open FStar.Stubs.Reflection.Types
open FStar.Stubs.Syntax.Syntax

(* V1 does not really use the primitive ident type, but this
explicit pair of string & range *)
Expand Down
8 changes: 8 additions & 0 deletions ulib/FStar.Stubs.Syntax.Syntax.fsti
Original file line number Diff line number Diff line change
Expand Up @@ -10,3 +10,11 @@ type subst_elt =
| UN : int -> universe -> subst_elt
| UD : ident -> int -> subst_elt
type subst_t = list subst_elt


(*
* match e as binder returns t|C
*
* the bool says whether returns (bool = false) or returns$ (bool = true, use type equality
*)
type match_returns_ascription = binder & (either term comp & option term & bool)

0 comments on commit 9ec5695

Please sign in to comment.