diff options
| author | Guillaume Melquiond | 2015-12-07 10:52:14 +0100 |
|---|---|---|
| committer | Guillaume Melquiond | 2015-12-07 10:52:24 +0100 |
| commit | df3a49a18c5b01984000df9244ecea9c275b30cd (patch) | |
| tree | d14afdb5de5f93e4301f8eba8bddecd5a6597f9a /theories/Structures | |
| parent | fe2776f9e0d355cccb0841495a9843351d340066 (diff) | |
Fix some typos.
Diffstat (limited to 'theories/Structures')
| -rw-r--r-- | theories/Structures/EqualitiesFacts.v | 2 | ||||
| -rw-r--r-- | theories/Structures/OrderedType.v | 2 | ||||
| -rw-r--r-- | theories/Structures/OrdersLists.v | 2 |
3 files changed, 3 insertions, 3 deletions
diff --git a/theories/Structures/EqualitiesFacts.v b/theories/Structures/EqualitiesFacts.v index 8e2b2d081c..d5827d87a0 100644 --- a/theories/Structures/EqualitiesFacts.v +++ b/theories/Structures/EqualitiesFacts.v @@ -60,7 +60,7 @@ Module KeyDecidableType(D:DecidableType). Hint Resolve eqke_1 eqke_2 eqk_1. - (* Additionnal facts *) + (* Additional facts *) Lemma InA_eqke_eqk {elt} p (m:list (key*elt)) : InA eqke p m -> InA eqk p m. diff --git a/theories/Structures/OrderedType.v b/theories/Structures/OrderedType.v index cc8c2261b6..93ca383b28 100644 --- a/theories/Structures/OrderedType.v +++ b/theories/Structures/OrderedType.v @@ -342,7 +342,7 @@ Module KeyOrderedType(O:OrderedType). compute in Hxx'; compute in Hyy'. rewrite Hxx', Hyy'; auto. Qed. - (* Additionnal facts *) + (* Additional facts *) Lemma eqk_not_ltk : forall x x', eqk x x' -> ~ltk x x'. Proof. diff --git a/theories/Structures/OrdersLists.v b/theories/Structures/OrdersLists.v index 4d49ac84ed..41e65d7287 100644 --- a/theories/Structures/OrdersLists.v +++ b/theories/Structures/OrdersLists.v @@ -76,7 +76,7 @@ Module KeyOrderedType(O:OrderedType). Instance ltk_compat' {elt} : Proper (eqke==>eqke==>iff) (@ltk elt). Proof. eapply subrelation_proper; eauto with *. Qed. - (* Additionnal facts *) + (* Additional facts *) Instance pair_compat {elt} : Proper (O.eq==>Logic.eq==>eqke) (@pair key elt). Proof. apply pair_compat. Qed. |
