From 9b01e3d8567122d5494b33ce3b8ce6e8eaf9a109 Mon Sep 17 00:00:00 2001
From: Robbert Krebbers <mail@robbertkrebbers.nl>
Date: Tue, 30 May 2017 23:43:15 +0200
Subject: [PATCH] Fix some spacing.

---
 theories/decidable.v | 8 ++++----
 1 file changed, 4 insertions(+), 4 deletions(-)

diff --git a/theories/decidable.v b/theories/decidable.v
index 52c7bc41..cb6213ad 100644
--- a/theories/decidable.v
+++ b/theories/decidable.v
@@ -37,10 +37,10 @@ Lemma decide_iff {A} P Q `{Decision P, Decision Q} (x y : A) :
   (P ↔ Q) → (if decide P then x else y) = (if decide Q then x else y).
 Proof. intros [??]. destruct (decide P), (decide Q); tauto. Qed.
 
-Lemma decide_left`{Decision P, !ProofIrrel P} (HP : P) : decide P = left HP.
-Proof. destruct (decide P) as [?|?]; [|contradiction]. f_equal. apply proof_irrel. Qed.
-Lemma decide_right`{Decision P} `{!ProofIrrel (¬ P)} (HP : ¬ P) : decide P = right HP.
-Proof. destruct (decide P) as [?|?]; [contradiction|]. f_equal. apply proof_irrel. Qed.
+Lemma decide_left `{Decision P, !ProofIrrel P} (HP : P) : decide P = left HP.
+Proof. destruct (decide P); [|contradiction]. f_equal. apply proof_irrel. Qed.
+Lemma decide_right `{Decision P, !ProofIrrel (¬ P)} (HP : ¬ P) : decide P = right HP.
+Proof. destruct (decide P); [contradiction|]. f_equal. apply proof_irrel. Qed.
 
 (** The tactic [destruct_decide] destructs a sumbool [dec]. If one of the
 components is double negated, it will try to remove the double negation. *)
-- 
GitLab