-
Notifications
You must be signed in to change notification settings - Fork 5
/
iota_reduction_fact8.v
29 lines (23 loc) · 1.15 KB
/
iota_reduction_fact8.v
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
16
17
18
19
20
21
22
23
24
25
26
27
28
29
Require Import PerformanceExperiments.Harness.
Require Export PerformanceExperiments.iota_reduction_common.
Global Open Scope Z_scope.
Local Notation factn := 8.
Local Notation with_abstract := false.
Definition args_of_size (s : size) : list Z
:= match s with
| Sanity => List.map Z.of_nat (seq 0 3)
| SuperFast => List.map (fun x => Z.of_nat x * 100) (seq 1 10)
| Fast => List.map (fun x => Z.of_nat x * 100) (seq 1 200)
| Medium => []
| Slow => []
| VerySlow => []
end.
Ltac describe_goal0 n := describe_goal_gen constr:(factn) slow n.
Ltac time_solve_goal0 n v := time_solve_goal_gen_slow constr:(with_abstract) n v.
Ltac run0 sz := idtac; Harness.runtests_step_constr args_of_size describe_goal0 step_goal_constr redgoal_constr time_solve_goal0 sz ltac:(mkgoal_init slow constr:(factn)).
Ltac describe_goal1 n := describe_goal_gen constr:(factn) fast n.
Ltac time_solve_goal1 n v := time_solve_goal_gen_fast constr:(with_abstract) n v.
Ltac run1 sz := Harness.runtests_step_constr args_of_size describe_goal1 step_goal_constr redgoal_constr time_solve_goal1 sz ltac:(mkgoal_init fast constr:(factn)).
(*
Goal True. run0 Fast.
*)