Skip to content

Commit

Permalink
[chore] update to follow main
Browse files Browse the repository at this point in the history
  • Loading branch information
fdupress committed Dec 8, 2023
1 parent 0c9e84d commit 4801702
Showing 1 changed file with 0 additions and 5 deletions.
5 changes: 0 additions & 5 deletions sha3/proof/Common.ec
Original file line number Diff line number Diff line change
Expand Up @@ -11,9 +11,6 @@ pragma +implicits.
op r : { int | 2 <= r } as ge2_r.
op c : { int | 0 < c } as gt0_c.

type block. (* ~ bitstrings of size r *)
type capacity. (* ~ bitstrings of size c *)

(* -------------------------------------------------------------------- *)

lemma gt0_r : 0 < r.
Expand All @@ -27,7 +24,6 @@ proof. by apply/ltrW/gt0_c. qed.

(* -------------------------------------------------------------------- *)
clone export BitWord as Capacity with
type word <- capacity,
op n <- c
proof gt0_n by apply/gt0_c

Expand All @@ -38,7 +34,6 @@ clone export BitWord as Capacity with
export Capacity DCapacity.

clone export BitWord as Block with
type word <- block,
op n <- r
proof gt0_n by apply/gt0_r

Expand Down

0 comments on commit 4801702

Please sign in to comment.