aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Sets/Constructive_sets.v
diff options
context:
space:
mode:
Diffstat (limited to 'theories/Sets/Constructive_sets.v')
-rwxr-xr-xtheories/Sets/Constructive_sets.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/Sets/Constructive_sets.v b/theories/Sets/Constructive_sets.v
index 9d24ae433..78ad3d2f2 100755
--- a/theories/Sets/Constructive_sets.v
+++ b/theories/Sets/Constructive_sets.v
@@ -38,7 +38,7 @@ Qed.
Lemma Noone_in_empty: (x: U) ~ (In U (Empty_set U) x).
Proof.
-Intro x; Red; Induction 1.
+Red; NewDestruct 1.
Qed.
Hints Resolve Noone_in_empty.