aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Logic
diff options
context:
space:
mode:
Diffstat (limited to 'theories/Logic')
-rw-r--r--theories/Logic/ClassicalFacts.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/Logic/ClassicalFacts.v b/theories/Logic/ClassicalFacts.v
index f82b00a0d..d4ebfb42f 100644
--- a/theories/Logic/ClassicalFacts.v
+++ b/theories/Logic/ClassicalFacts.v
@@ -688,7 +688,7 @@ Section Unrestricted_minimization_entails_excluded_middle.
apply unrestricted_minimization in h as ([|[|m]] & hm & hmm).
+ intuition.
+ right.
- intros /p₀/hmm/PeanoNat.Nat.nle_succ_0-HA. assumption.
+ intros HA. apply p₀, hmm, PeanoNat.Nat.nle_succ_0 in HA. assumption.
+ destruct hm as [([=],_) | [=] ].
Qed.