Skip to content

Commit 540e6a2

Browse files
committed
Use Listable to prove equality of registers and opcodes
This is much faster, especially as we add more registers and opcodes
1 parent 3878d76 commit 540e6a2

11 files changed

+365
-266
lines changed

src/Assembly/Equality.v

+10-10
Original file line numberDiff line numberDiff line change
@@ -35,8 +35,8 @@ Bind Scope REG_scope with REG.
3535
Infix "=?" := REG_beq : REG_scope.
3636

3737
Global Instance REG_beq_spec : reflect_rel (@eq REG) REG_beq | 10
38-
:= reflect_of_beq internal_REG_dec_bl internal_REG_dec_lb.
39-
Definition REG_beq_eq x y : (x =? y)%REG = true <-> x = y := conj (@internal_REG_dec_bl _ _) (@internal_REG_dec_lb _ _).
38+
:= reflect_of_beq REG_dec_bl REG_dec_lb.
39+
Definition REG_beq_eq x y : (x =? y)%REG = true <-> x = y := conj (@REG_dec_bl _ _) (@REG_dec_lb _ _).
4040
Lemma REG_beq_neq x y : (x =? y)%REG = false <-> x <> y.
4141
Proof. rewrite <- REG_beq_eq; destruct (x =? y)%REG; intuition congruence. Qed.
4242
Global Instance REG_beq_compat : Proper (eq ==> eq ==> eq) REG_beq | 10.
@@ -95,8 +95,8 @@ Bind Scope AccessSize_scope with AccessSize.
9595
Infix "=?" := AccessSize_beq : AccessSize_scope.
9696

9797
Global Instance AccessSize_beq_spec : reflect_rel (@eq AccessSize) AccessSize_beq | 10
98-
:= reflect_of_beq internal_AccessSize_dec_bl internal_AccessSize_dec_lb.
99-
Definition AccessSize_beq_eq x y : (x =? y)%AccessSize = true <-> x = y := conj (@internal_AccessSize_dec_bl _ _) (@internal_AccessSize_dec_lb _ _).
98+
:= reflect_of_beq AccessSize_dec_bl AccessSize_dec_lb.
99+
Definition AccessSize_beq_eq x y : (x =? y)%AccessSize = true <-> x = y := conj (@AccessSize_dec_bl _ _) (@AccessSize_dec_lb _ _).
100100
Lemma AccessSize_beq_neq x y : (x =? y)%AccessSize = false <-> x <> y.
101101
Proof. rewrite <- AccessSize_beq_eq; destruct (x =? y)%AccessSize; intuition congruence. Qed.
102102
Global Instance AccessSize_beq_compat : Proper (eq ==> eq ==> eq) AccessSize_beq | 10.
@@ -141,8 +141,8 @@ Bind Scope FLAG_scope with FLAG.
141141
Infix "=?" := FLAG_beq : FLAG_scope.
142142

143143
Global Instance FLAG_beq_spec : reflect_rel (@eq FLAG) FLAG_beq | 10
144-
:= reflect_of_beq internal_FLAG_dec_bl internal_FLAG_dec_lb.
145-
Definition FLAG_beq_eq x y : (x =? y)%FLAG = true <-> x = y := conj (@internal_FLAG_dec_bl _ _) (@internal_FLAG_dec_lb _ _).
144+
:= reflect_of_beq FLAG_dec_bl FLAG_dec_lb.
145+
Definition FLAG_beq_eq x y : (x =? y)%FLAG = true <-> x = y := conj (@FLAG_dec_bl _ _) (@FLAG_dec_lb _ _).
146146
Lemma FLAG_beq_neq x y : (x =? y)%FLAG = false <-> x <> y.
147147
Proof. rewrite <- FLAG_beq_eq; destruct (x =? y)%FLAG; intuition congruence. Qed.
148148
Global Instance FLAG_beq_compat : Proper (eq ==> eq ==> eq) FLAG_beq | 10.
@@ -155,8 +155,8 @@ Bind Scope OpCode_scope with OpCode.
155155
Infix "=?" := OpCode_beq : OpCode_scope.
156156

157157
Global Instance OpCode_beq_spec : reflect_rel (@eq OpCode) OpCode_beq | 10
158-
:= reflect_of_beq internal_OpCode_dec_bl internal_OpCode_dec_lb.
159-
Definition OpCode_beq_eq x y : (x =? y)%OpCode = true <-> x = y := conj (@internal_OpCode_dec_bl _ _) (@internal_OpCode_dec_lb _ _).
158+
:= reflect_of_beq OpCode_dec_bl OpCode_dec_lb.
159+
Definition OpCode_beq_eq x y : (x =? y)%OpCode = true <-> x = y := conj (@OpCode_dec_bl _ _) (@OpCode_dec_lb _ _).
160160
Lemma OpCode_beq_neq x y : (x =? y)%OpCode = false <-> x <> y.
161161
Proof. rewrite <- OpCode_beq_eq; destruct (x =? y)%OpCode; intuition congruence. Qed.
162162
Global Instance OpCode_beq_compat : Proper (eq ==> eq ==> eq) OpCode_beq | 10.
@@ -169,8 +169,8 @@ Bind Scope OpPrefix_scope with OpPrefix.
169169
Infix "=?" := OpPrefix_beq : OpPrefix_scope.
170170

171171
Global Instance OpPrefix_beq_spec : reflect_rel (@eq OpPrefix) OpPrefix_beq | 10
172-
:= reflect_of_beq internal_OpPrefix_dec_bl internal_OpPrefix_dec_lb.
173-
Definition OpPrefix_beq_eq x y : (x =? y)%OpPrefix = true <-> x = y := conj (@internal_OpPrefix_dec_bl _ _) (@internal_OpPrefix_dec_lb _ _).
172+
:= reflect_of_beq OpPrefix_dec_bl OpPrefix_dec_lb.
173+
Definition OpPrefix_beq_eq x y : (x =? y)%OpPrefix = true <-> x = y := conj (@OpPrefix_dec_bl _ _) (@OpPrefix_dec_lb _ _).
174174
Lemma OpPrefix_beq_neq x y : (x =? y)%OpPrefix = false <-> x <> y.
175175
Proof. rewrite <- OpPrefix_beq_eq; destruct (x =? y)%OpPrefix; intuition congruence. Qed.
176176
Global Instance OpPrefix_beq_compat : Proper (eq ==> eq ==> eq) OpPrefix_beq | 10.

src/Assembly/Equivalence.v

+2-2
Original file line numberDiff line numberDiff line change
@@ -1275,10 +1275,10 @@ Definition init_symbolic_state_descr : description := Build_description "init_sy
12751275

12761276
Definition init_symbolic_state (d : dag) : symbolic_state
12771277
:= let _ := init_symbolic_state_descr in
1278-
let '(initial_reg_idxs, d) := dag_gensym_n 16 d in
1278+
let '(initial_reg_idxs, d) := dag_gensym_n (List.length widest_registers) d in
12791279
{|
12801280
dag_state := d;
1281-
symbolic_reg_state := Tuple.from_list_default None 16 (List.map Some initial_reg_idxs);
1281+
symbolic_reg_state := Tuple.from_list_default None _ (List.map Some initial_reg_idxs);
12821282
symbolic_mem_state := [];
12831283
symbolic_flag_state := Tuple.repeat None 6;
12841284
|}.

src/Assembly/EquivalenceProofs.v

+2-2
Original file line numberDiff line numberDiff line change
@@ -1847,7 +1847,7 @@ Qed.
18471847
(* TODO: this is Symbolic.get_reg; move to SymbolicProofs? *)
18481848
Lemma get_reg_set_reg_full s rn rn' v
18491849
: get_reg (set_reg s rn v) rn'
1850-
= if ((rn <? ((fun n (_ : Tuple.tuple _ n) => n) _ s)) && (rn =? rn'))%nat%bool
1850+
= if ((rn <? ((fun n (_ : Tuple.tuple _ n) => N.of_nat n) _ s)) && (rn =? rn'))%N%bool
18511851
then Some v
18521852
else get_reg s rn'.
18531853
Proof.
@@ -1863,7 +1863,7 @@ Qed.
18631863

18641864
(* TODO: this is Symbolic.get_reg; move to SymbolicProofs? *)
18651865
Local Lemma get_reg_set_reg_same s rn v
1866-
(H : (rn < (fun n (_ : Tuple.tuple _ n) => n) _ s)%nat)
1866+
(H : (rn < (fun n (_ : Tuple.tuple _ n) => N.of_nat n) _ s)%N)
18671867
: get_reg (set_reg s rn v) rn = Some v.
18681868
Proof.
18691869
rewrite get_reg_set_reg_full; break_innermost_match; reflect_hyps; cbv beta in *; try reflexivity; lia.

src/Assembly/Parse.v

-20
Original file line numberDiff line numberDiff line change
@@ -22,34 +22,18 @@ Local Open Scope list_scope.
2222
Local Open Scope string_scope.
2323
Local Open Scope parse_scope.
2424

25-
Derive REG_Listable SuchThat (@FinitelyListable REG REG_Listable) As REG_FinitelyListable.
26-
Proof. prove_ListableDerive. Qed.
27-
Global Existing Instances REG_Listable REG_FinitelyListable.
28-
2925
Global Instance show_REG : Show REG.
3026
Proof. prove_Show_enum (). Defined.
3127
Global Instance show_lvl_REG : ShowLevel REG := show_REG.
3228

33-
Derive FLAG_Listable SuchThat (@FinitelyListable FLAG FLAG_Listable) As FLAG_FinitelyListable.
34-
Proof. prove_ListableDerive. Qed.
35-
Global Existing Instances FLAG_Listable FLAG_FinitelyListable.
36-
3729
Global Instance show_FLAG : Show FLAG.
3830
Proof. prove_Show_enum (). Defined.
3931
Global Instance show_lvl_FLAG : ShowLevel FLAG := show_FLAG.
4032

41-
Derive OpCode_Listable SuchThat (@FinitelyListable OpCode OpCode_Listable) As OpCode_FinitelyListable.
42-
Proof. prove_ListableDerive. Qed.
43-
Global Existing Instances OpCode_Listable OpCode_FinitelyListable.
44-
4533
Global Instance show_OpCode : Show OpCode.
4634
Proof. prove_Show_enum (). Defined.
4735
Global Instance show_lvl_OpCode : ShowLevel OpCode := show_OpCode.
4836

49-
Derive OpPrefix_Listable SuchThat (@FinitelyListable OpPrefix OpPrefix_Listable) As OpPrefix_FinitelyListable.
50-
Proof. prove_ListableDerive. Qed.
51-
Global Existing Instances OpPrefix_Listable OpPrefix_FinitelyListable.
52-
5337
Global Instance show_OpPrefix : Show OpPrefix.
5438
Proof. prove_Show_enum (). Defined.
5539
Global Instance show_lvl_OpPrefix : ShowLevel OpPrefix := show_OpPrefix.
@@ -72,10 +56,6 @@ Definition parse_FLAG_list : list (string * FLAG)
7256
Definition parse_FLAG : ParserAction FLAG
7357
:= parse_strs parse_FLAG_list.
7458

75-
Derive AccessSize_Listable SuchThat (@FinitelyListable AccessSize AccessSize_Listable) As AccessSize_FinitelyListable.
76-
Proof. prove_ListableDerive. Qed.
77-
Global Existing Instances AccessSize_Listable AccessSize_FinitelyListable.
78-
7959
Global Instance show_AccessSize : Show AccessSize.
8060
Proof. prove_Show_enum (). Defined.
8161
Global Instance show_lvl_AccessSize : ShowLevel AccessSize := show_AccessSize.

src/Assembly/Symbolic.v

+10-10
Original file line numberDiff line numberDiff line change
@@ -3829,7 +3829,7 @@ Definition simplify {opts : symbolic_options_computed_opt} (dag : dag) (e : node
38293829
Lemma eval_simplify {opts : symbolic_options_computed_opt} G d n v : gensym_dag_ok G d -> eval_node G d n v -> eval G d (simplify d n) v.
38303830
Proof using Type. eauto using Rewrite.eval_expr, eval_node_reveal_node_at_least. Qed.
38313831

3832-
Definition reg_state := Tuple.tuple (option idx) 16.
3832+
Definition reg_state := Tuple.tuple (option idx) (compute! (List.length widest_registers)).
38333833
Definition flag_state := Tuple.tuple (option idx) 6.
38343834
Definition mem_state := list (idx * idx).
38353835

@@ -3863,16 +3863,16 @@ Definition reverse_lookup_flag (st : flag_state) (i : idx) : option FLAG
38633863
(List.find (fun v => option_beq N.eqb (Some i) (fst v))
38643864
(Tuple.to_list _ (Tuple.map2 (@pair _ _) st (CF, PF, AF, ZF, SF, OF)))).
38653865

3866-
Definition get_reg (st : reg_state) (ri : nat) : option idx
3867-
:= Tuple.nth_default None ri st.
3868-
Definition set_reg (st : reg_state) ri (i : idx) : reg_state
3866+
Definition get_reg (st : reg_state) (ri : N) : option idx
3867+
:= Tuple.nth_default None (N.to_nat ri) st.
3868+
Definition set_reg (st : reg_state) (ri : N) (i : idx) : reg_state
38693869
:= Tuple.from_list_default None _ (ListUtil.set_nth
3870-
ri
3870+
(N.to_nat ri)
38713871
(Some i)
38723872
(Tuple.to_list _ st)).
38733873
Definition reverse_lookup_widest_reg (st : reg_state) (i : idx) : option REG
38743874
:= option_map
3875-
(fun v => widest_register_of_index (fst v))
3875+
(fun v => widest_register_of_index (N.of_nat (fst v)))
38763876
(List.find (fun v => option_beq N.eqb (Some i) (snd v))
38773877
(List.enumerate (Tuple.to_list _ st))).
38783878

@@ -3906,7 +3906,7 @@ Definition update_mem_with (st : symbolic_state) (f : mem_state -> mem_state) :
39063906
:= {| dag_state := st.(dag_state); symbolic_reg_state := st.(symbolic_reg_state) ; symbolic_flag_state := st.(symbolic_flag_state) ; symbolic_mem_state := f st.(symbolic_mem_state) |}.
39073907

39083908
Global Instance show_reg_state : Show reg_state := fun st =>
3909-
show (List.map (fun '(n, v) => (widest_register_of_index n, v)) (ListUtil.List.enumerate (Option.List.map id (Tuple.to_list _ st)))).
3909+
show (List.combine widest_registers (Option.List.map id (Tuple.to_list _ st))).
39103910

39113911
Global Instance show_flag_state : Show flag_state :=
39123912
fun '(cfv, pfv, afv, zfv, sfv, ofv) => (
@@ -3953,7 +3953,7 @@ Module error.
39533953
Local Unset Decidable Equality Schemes.
39543954
Variant error :=
39553955
| get_flag (f : FLAG) (s : flag_state)
3956-
| get_reg (r : nat + REG) (s : reg_state)
3956+
| get_reg (r : N + REG) (s : reg_state)
39573957
| load (a : idx) (s : symbolic_state)
39583958
| remove (a : idx) (s : symbolic_state)
39593959
| remove_has_duplicates (a : idx) (vs : list idx) (s : symbolic_state)
@@ -3977,7 +3977,7 @@ Module error.
39773977
=> ["In flag state " ++ show_flag_state s;
39783978
"Flag " ++ show f ++ " was read without being set."]
39793979
| get_reg (inl i) s
3980-
=> ["Invalid reg index " ++ show_nat i]
3980+
=> ["Invalid reg index " ++ show i]
39813981
| get_reg (inr r) s
39823982
=> ["In reg state " ++ show_reg_state s;
39833983
"Register " ++ show (r : REG) ++ " read without being set."]
@@ -4042,7 +4042,7 @@ Definition mapM_ {A B} (f: A -> M B) l : M unit := _ <- mapM f l; ret tt.
40424042

40434043
Definition error_get_reg_of_reg_index ri : symbolic_state -> error
40444044
:= error.get_reg (let r := widest_register_of_index ri in
4045-
if (reg_index r =? ri)%nat
4045+
if (reg_index r =? ri)%N
40464046
then inr r
40474047
else inl ri).
40484048

0 commit comments

Comments
 (0)