Skip to content

Commit 67e65e8

Browse files
authored
Merge pull request #3924 from mtzguido/tactics
Tactics: make V2 the default
2 parents 373c46b + b753caf commit 67e65e8

16 files changed

+26
-25
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

ulib/FStar.Reflection.Formula.fst

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -16,4 +16,4 @@
1616
module FStar.Reflection.Formula
1717

1818
(* This module is a temporary for Meta-F* migration *)
19-
include FStar.Reflection.V1.Formula
19+
include FStar.Reflection.V2.Formula

ulib/FStar.Reflection.fst

Lines changed: 3 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -15,6 +15,6 @@
1515
*)
1616
module FStar.Reflection
1717

18-
(* This switch currently points to V1. Ask for V2 explicitly by
19-
importing FStar.Reflection.V2 *)
20-
include FStar.Reflection.V1
18+
(* This switch currently points to V2. Ask for V1 explicitly by
19+
importing FStar.Reflection.V1 *)
20+
include FStar.Reflection.V2

ulib/FStar.Tactics.Builtins.fsti

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -16,4 +16,4 @@
1616
module FStar.Tactics.Builtins
1717

1818
(* This module is a temporary for Meta-F* migration *)
19-
include FStar.Stubs.Tactics.V1.Builtins
19+
include FStar.Stubs.Tactics.V2.Builtins

ulib/FStar.Tactics.Derived.fst

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -16,4 +16,4 @@
1616
module FStar.Tactics.Derived
1717

1818
(* This module is a temporary for Meta-F* migration *)
19-
include FStar.Tactics.V1.Derived
19+
include FStar.Tactics.V2.Derived

ulib/FStar.Tactics.Logic.fst

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -16,4 +16,4 @@
1616
module FStar.Tactics.Logic
1717

1818
(* This module is a temporary for Meta-F* migration *)
19-
include FStar.Tactics.V1.Logic
19+
include FStar.Tactics.V2.Logic

ulib/FStar.Tactics.SyntaxHelpers.fst

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -16,4 +16,4 @@
1616
module FStar.Tactics.SyntaxHelpers
1717

1818
(* This module is a temporary for Meta-F* migration *)
19-
include FStar.Tactics.V1.SyntaxHelpers
19+
include FStar.Tactics.V2.SyntaxHelpers

ulib/FStar.Tactics.V2.Logic.fsti

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -21,7 +21,7 @@ open FStar.Reflection.V2.Formula
2121
open FStar.Tactics.NamedView
2222
open FStar.Tactics.Logic.Lemmas {} (* bring lemmas into TC scope *)
2323

24-
(* Repeated to avoid importing FStar.Tactics.V1.Derived. *)
24+
(* Repeated to avoid importing FStar.Tactics.Derived. *)
2525
private let cur_goal () : Tac typ =
2626
let open FStar.Stubs.Tactics.Types in
2727
let open FStar.Stubs.Tactics.V2.Builtins in

ulib/FStar.Tactics.fsti

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -15,4 +15,4 @@
1515
*)
1616
module FStar.Tactics
1717

18-
include FStar.Tactics.V1
18+
include FStar.Tactics.V2

0 commit comments

Comments
 (0)