aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Init/Logic.v
diff options
context:
space:
mode:
authorGravatar Vadim Zaliva <lord@crocodile.org>2017-04-26 11:21:10 -0700
committerGravatar GitHub <noreply@github.com>2017-04-26 11:21:10 -0700
commit2fc235b0e00c028d2e91c696926ad339232d51e3 (patch)
tree5aac50c21c08138256f5800c6daf68357326a6ba /theories/Init/Logic.v
parentadc2035410a339cfa88dae527b631f5131adaa54 (diff)
Small typo in comment
Diffstat (limited to 'theories/Init/Logic.v')
-rw-r--r--theories/Init/Logic.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/Init/Logic.v b/theories/Init/Logic.v
index f659c31f9..9ae9dde28 100644
--- a/theories/Init/Logic.v
+++ b/theories/Init/Logic.v
@@ -223,7 +223,7 @@ Proof.
Qed.
(** [(IF_then_else P Q R)], written [IF P then Q else R] denotes
- either [P] and [Q], or [~P] and [Q] *)
+ either [P] and [Q], or [~P] and [R] *)
Definition IF_then_else (P Q R:Prop) := P /\ Q \/ ~ P /\ R.