diff options
| author | Hugo Herbelin | 2020-04-08 19:18:55 +0200 |
|---|---|---|
| committer | Hugo Herbelin | 2020-04-08 19:18:55 +0200 |
| commit | 459faeddd095789affa30e7cf3b59fdaf95c1a0f (patch) | |
| tree | b4d1d96023e0729d6cf06f77f4e2b4e7522f4f7a /theories/Numbers | |
| parent | b26d1f477990d88e235ffda0f23f494456ce5862 (diff) | |
| parent | 50a55c0c6eac87a6aaf281dba9b2bc5b0359b09d (diff) | |
Merge PR #11909: Make the level of ≡ in Int63 consistent with =
Reviewed-by: anton-trunov
Diffstat (limited to 'theories/Numbers')
| -rw-r--r-- | theories/Numbers/Cyclic/Int63/Int63.v | 2 |
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/Numbers/Cyclic/Int63/Int63.v b/theories/Numbers/Cyclic/Int63/Int63.v index c4f738ac39..bacc4a7650 100644 --- a/theories/Numbers/Cyclic/Int63/Int63.v +++ b/theories/Numbers/Cyclic/Int63/Int63.v @@ -690,7 +690,7 @@ Proof. now intros h; rewrite (to_Z_inj _ 0 h). Qed. Lemma tail00_spec x : φ x = 0 -> φ (tail0 x) = φ digits. Proof. now intros h; rewrite (to_Z_inj _ 0 h). Qed. -Infix "≡" := (eqm wB) (at level 80) : int63_scope. +Infix "≡" := (eqm wB) (at level 70, no associativity) : int63_scope. Lemma eqm_mod x y : x mod wB ≡ y mod wB → x ≡ y. Proof. |
