Skip to content

Commit

Permalink
Merge pull request #747 from proux01/coq_18164
Browse files Browse the repository at this point in the history
Adapt to coq/coq#18164
  • Loading branch information
andrew-appel committed Nov 27, 2023
2 parents 8633963 + c1e7f88 commit 6d2eb96
Show file tree
Hide file tree
Showing 2 changed files with 1 addition and 3 deletions.
2 changes: 1 addition & 1 deletion floyd/reptype_lemmas.v
Original file line number Diff line number Diff line change
Expand Up @@ -1183,7 +1183,7 @@ change 0 with (Z.of_nat 0).
rewrite Zlength_correct.
rewrite replist_firstn_skipn by lia.
rewrite skipn_0 by auto.
rewrite NPeano.Nat.sub_0_r.
rewrite Nat.sub_0_r.
apply firstn_exact_length.
Qed.

Expand Down
2 changes: 0 additions & 2 deletions msl/tree_shares.v
Original file line number Diff line number Diff line change
Expand Up @@ -10,9 +10,7 @@ Require Import VST.msl.sepalg.
Require Import VST.msl.boolean_alg.

Require Import Recdef.
Require Import NPeano.
Require Import ZArith.
Require Import Coq.Arith.Max.

(** This module implements a share model
via binary trees with boolean-labeled leaves.
Expand Down

0 comments on commit 6d2eb96

Please sign in to comment.