Skip to content

Commit 62eb294

Browse files
committed
fixed wrong word
1 parent 29825b0 commit 62eb294

File tree

2 files changed

+2
-2
lines changed

2 files changed

+2
-2
lines changed

exercises/spin_lock.v

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -201,7 +201,7 @@ Definition prog : expr :=
201201

202202
(**
203203
[x] can take on the values of [0], [1], and [7]. However, we should
204-
not observe [7], as it is overridden before the lock is released.
204+
not observe [7], as it is overwritten before the lock is released.
205205
*)
206206
Lemma prog_spec : ⊢ WP prog {{ v, ⌜v = #0 ∨ v = #1⌝}}.
207207
Proof.

theories/spin_lock.v

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -210,7 +210,7 @@ Definition prog : expr :=
210210

211211
(**
212212
[x] can take on the values of [0], [1], and [7]. However, we should
213-
not observe [7], as it is overridden before the lock is released.
213+
not observe [7], as it is overwritten before the lock is released.
214214
*)
215215
Lemma prog_spec : ⊢ WP prog {{ v, ⌜v = #0 ∨ v = #1⌝}}.
216216
Proof.

0 commit comments

Comments
 (0)