aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Logic
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2015-12-05 10:21:33 +0100
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2015-12-05 10:23:05 +0100
commitb7e72d0e0ca64168fc16875bf779dbc27d2a1820 (patch)
tree1501dea5e28b1a07d998f6d8bfa52d4d5770ddbd /theories/Logic
parent6b39f9904b4e9d5260c4fd97ff10e52c489c6051 (diff)
Fix to previous commit (ClassicalFacts.v).
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.