aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Sets/Relations_2_facts.v
diff options
context:
space:
mode:
Diffstat (limited to 'theories/Sets/Relations_2_facts.v')
-rw-r--r--theories/Sets/Relations_2_facts.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/Sets/Relations_2_facts.v b/theories/Sets/Relations_2_facts.v
index 13ec1e6c4..89b98c1f5 100644
--- a/theories/Sets/Relations_2_facts.v
+++ b/theories/Sets/Relations_2_facts.v
@@ -148,4 +148,4 @@ elim (H'3 t); auto with sets.
intros z1 H'5; elim H'5; intros H'8 H'10; try exact H'8; clear H'5.
exists z1; split; [ idtac | assumption ].
apply Rstar_n with t; auto with sets.
-Qed. \ No newline at end of file
+Qed.