aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/IntMap/Adist.v
diff options
context:
space:
mode:
Diffstat (limited to 'theories/IntMap/Adist.v')
-rw-r--r--theories/IntMap/Adist.v3
1 files changed, 2 insertions, 1 deletions
diff --git a/theories/IntMap/Adist.v b/theories/IntMap/Adist.v
index f5d40e66f..4e545af7b 100644
--- a/theories/IntMap/Adist.v
+++ b/theories/IntMap/Adist.v
@@ -59,7 +59,8 @@ Proof.
Qed.
Lemma ad_plength_first_one : (a:ad) (n:nat)
- ((k:nat) (lt k n) -> (ad_bit a k)=false) -> (ad_bit a n)=true -> (ad_plength a)=(ni n).
+ ((k:nat) (lt k n) -> (ad_bit a k)=false) -> (ad_bit a n)=true
+ -> (ad_plength a)=(ni n).
Proof.
Induction a. Intros. Simpl in H0. Discriminate H0.
Induction p. Intros. Generalize H0. Case n. Intros. Reflexivity.