Skip to content

Commit

Permalink
bump coqutil
Browse files Browse the repository at this point in the history
and adapt to rewrite bug that got exposed by not importing Word
  • Loading branch information
samuelgruetter committed Apr 5, 2024
1 parent 4421d54 commit 75c4008
Show file tree
Hide file tree
Showing 3 changed files with 7 additions and 2 deletions.
3 changes: 2 additions & 1 deletion compiler/src/compiler/memory_mapped_ext_calls_compiler.v
Original file line number Diff line number Diff line change
Expand Up @@ -520,7 +520,8 @@ Section MMIO.
- eapply map.disjoint_putmany_l. split. 1: assumption.
apply map.disjoint_comm. assumption. }
{ cbn. rewrite word.unsigned_of_Z_nowrap by lia.
rewrite LittleEndian.split_combine. assumption. }
replace (LittleEndian.split n (LittleEndian.combine n v)) with v.
1: assumption. symmetry. apply LittleEndian.split_combine. }
lazymatch goal with
| HO: outcome _ _, H: forall _ _, outcome _ _ -> _ |- _ =>
specialize H with (1 := HO); destruct H as (l' & Hp & HPost)
Expand Down
4 changes: 4 additions & 0 deletions processor/src/processor/KamiRiscvStep.v
Original file line number Diff line number Diff line change
Expand Up @@ -38,6 +38,10 @@ Require Import processor.Consistency.

Local Open Scope Z_scope.

(* workaround for `rewrite` bug:
https://github.com/coq/coq/issues/1811#issuecomment-1320064508 *)
Local Set Keyed Unification.

Local Ltac subst_after_destr H ::= idtac.

(** Consistency between the Kami word and the Z-based word *)
Expand Down

0 comments on commit 75c4008

Please sign in to comment.