Skip to content

Commit

Permalink
Merge remote-tracking branch 'origin/master' into nik_restrict_inject…
Browse files Browse the repository at this point in the history
…ivity
  • Loading branch information
nikswamy committed Apr 19, 2024
2 parents db285db + 2c0ac7c commit 2aec69e
Show file tree
Hide file tree
Showing 23 changed files with 1,358 additions and 532 deletions.
56 changes: 26 additions & 30 deletions ocaml/fstar-lib/FStar_Tactics_V2_Builtins.ml
Original file line number Diff line number Diff line change
Expand Up @@ -34,35 +34,31 @@ let to_tac_1 (t: 'b -> 'a __tac): 'b -> 'a TM.tac = fun x ->
(fun (ps: proofstate) ->
uninterpret_tac (t x) ps) |> TM.mk_tac

let from_tac_1 s (t: 'a -> 'b TM.tac): 'a -> 'b __tac =
fun (x: 'a) ->
fun (ps: proofstate) ->
let m = t x in
interpret_tac s m ps

let from_tac_2 s (t: 'a -> 'b -> 'c TM.tac): 'a -> 'b -> 'c __tac =
fun (x: 'a) ->
fun (y: 'b) ->
fun (ps: proofstate) ->
let m = t x y in
interpret_tac s m ps

let from_tac_3 s (t: 'a -> 'b -> 'c -> 'd TM.tac): 'a -> 'b -> 'c -> 'd __tac =
fun (x: 'a) ->
fun (y: 'b) ->
fun (z: 'c) ->
fun (ps: proofstate) ->
let m = t x y z in
interpret_tac s m ps

let from_tac_4 s (t: 'a -> 'b -> 'c -> 'd -> 'e TM.tac): 'a -> 'b -> 'c -> 'd -> 'e __tac =
fun (x: 'a) ->
fun (y: 'b) ->
fun (z: 'c) ->
fun (w: 'd) ->
fun (ps: proofstate) ->
let m = t x y z w in
interpret_tac s m ps
let from_tac_1 s (t: 'a -> 'r TM.tac): 'a -> 'r __tac =
fun (xa: 'a) (ps : proofstate) ->
let m = t xa in
interpret_tac s m ps

let from_tac_2 s (t: 'a -> 'b -> 'r TM.tac): 'a -> 'b -> 'r __tac =
fun (xa: 'a) (xb: 'b) (ps : proofstate) ->
let m = t xa xb in
interpret_tac s m ps

let from_tac_3 s (t: 'a -> 'b -> 'c -> 'r TM.tac): 'a -> 'b -> 'c -> 'r __tac =
fun (xa: 'a) (xb: 'b) (xc: 'c) (ps : proofstate) ->
let m = t xa xb xc in
interpret_tac s m ps

let from_tac_4 s (t: 'a -> 'b -> 'c -> 'd -> 'r TM.tac): 'a -> 'b -> 'c -> 'd -> 'r __tac =
fun (xa: 'a) (xb: 'b) (xc: 'c) (xd: 'd) (ps : proofstate) ->
let m = t xa xb xc xd in
interpret_tac s m ps

let from_tac_5 s (t: 'a -> 'b -> 'c -> 'd -> 'e -> 'r TM.tac): 'a -> 'b -> 'c -> 'd -> 'e -> 'r __tac =
fun (xa: 'a) (xb: 'b) (xc: 'c) (xd: 'd) (xe: 'e) (ps : proofstate) ->
let m = t xa xb xc xd xe in
interpret_tac s m ps


(* Pointing to the internal primitives *)
let compress = from_tac_1 "B.compress" B.compress
Expand Down Expand Up @@ -146,7 +142,7 @@ type ('env, 'sc, 't, 'pats, 'bnds) match_complete_token = unit

let is_non_informative = from_tac_2 "B.refl_is_non_informative" B.refl_is_non_informative
let check_subtyping = from_tac_3 "B.refl_check_subtyping" B.refl_check_subtyping
let check_equiv = from_tac_3 "B.refl_check_equiv" B.refl_check_equiv
let t_check_equiv = from_tac_5 "B.t_refl_check_equiv" B.t_refl_check_equiv
let core_compute_term_type = from_tac_2 "B.refl_core_compute_term_type" B.refl_core_compute_term_type
let core_check_term = from_tac_4 "B.refl_core_check_term" B.refl_core_check_term
let core_check_term_at_type = from_tac_3 "B.refl_core_check_term_at_type" B.refl_core_check_term_at_type
Expand Down
84 changes: 84 additions & 0 deletions ocaml/fstar-lib/generated/FStar_Tactics_InterpFuns.ml

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

2 changes: 1 addition & 1 deletion ocaml/fstar-lib/generated/FStar_Tactics_V1_Basic.ml

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

Loading

0 comments on commit 2aec69e

Please sign in to comment.