Skip to content

Commit 5b17fec

Browse files
committed
Update tests
1 parent e83f8e2 commit 5b17fec

File tree

2 files changed

+10
-9
lines changed

2 files changed

+10
-9
lines changed

tests/micro-benchmarks/Misc.Norm3.fst

Lines changed: 5 additions & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -8,6 +8,7 @@ will fail to typecheck. *)
88
open FStar.Ghost
99
open FStar.Tactics
1010
open FStar.Reflection.Typing
11+
module R = FStar.Reflection
1112

1213
[@@erasable]
1314
noeq
@@ -16,21 +17,21 @@ type my_erased (a:Type) = | E of a
1617
let test (r_env goal : _) : Tac unit =
1718
let u0 = pack_universe Uv_Zero in
1819
let goal_typing :
19-
my_erased (typing_token r_env goal (E_Total, pack_ln (Tv_Type u0)))
20+
my_erased (typing_token r_env goal (E_Total, pack_ln (R.Tv_Type u0)))
2021
= magic()
2122
in
22-
let goal_typing_tok : squash (typing_token r_env goal (E_Total, pack_ln (Tv_Type u0))) =
23+
let goal_typing_tok : squash (typing_token r_env goal (E_Total, pack_ln (R.Tv_Type u0))) =
2324
match goal_typing with E x -> ()
2425
in
2526
()
2627

2728
(* This should always work regardless of the comment above. *)
2829
let test2 (r_env goal u0 : _) : Tac unit =
2930
let goal_typing :
30-
my_erased (typing_token r_env goal (E_Total, pack_ln (Tv_Type u0)))
31+
my_erased (typing_token r_env goal (E_Total, pack_ln (R.Tv_Type u0)))
3132
= magic()
3233
in
33-
let goal_typing_tok : squash (typing_token r_env goal (E_Total, pack_ln (Tv_Type u0))) =
34+
let goal_typing_tok : squash (typing_token r_env goal (E_Total, pack_ln (R.Tv_Type u0))) =
3435
match goal_typing with E x -> ()
3536
in
3637
()

tests/tactics/NoDuplicateSplice.fst

Lines changed: 5 additions & 5 deletions
Original file line numberDiff line numberDiff line change
@@ -3,11 +3,11 @@ module NoDuplicateSplice
33
open FStar.Tactics
44

55
let mk (nm:string) (i:int) : Tac decls =
6-
let lb = pack_lb ({ lb_fv = pack_fv (cur_module() @ [nm])
7-
; lb_us = []
8-
; lb_typ = `int
9-
; lb_def = pack (Tv_Const (C_Int i)) }) in
10-
[pack_sigelt (Sg_Let false [lb])]
6+
let lb = { lb_fv = pack_fv (cur_module() @ [nm])
7+
; lb_us = []
8+
; lb_typ = `int
9+
; lb_def = pack (Tv_Const (C_Int i)) } in
10+
[pack_sigelt (Sg_Let {isrec=false; lbs=[lb]})]
1111

1212
%splice[] (mk "x" 1)
1313

0 commit comments

Comments
 (0)