diff options
| author | coqbot-app[bot] | 2021-04-21 14:58:51 +0000 |
|---|---|---|
| committer | GitHub | 2021-04-21 14:58:51 +0000 |
| commit | f9996cdaf0b6aee12c5b71432b1edb90dffb569a (patch) | |
| tree | 99bacd74ac72db0aed31f18280b08be3db794db2 /theories/Classes/SetoidDec.v | |
| parent | 3645c06030ed1266fd4160ec7211b4447731bf13 (diff) | |
| parent | eeb142f3c69d2467fbadd7dd1470ac1606b2e5bf (diff) | |
Merge PR #13911: Remove the :> type cast?
Reviewed-by: mattam82
Ack-by: Zimmi48
Diffstat (limited to 'theories/Classes/SetoidDec.v')
| -rw-r--r-- | theories/Classes/SetoidDec.v | 2 |
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/Classes/SetoidDec.v b/theories/Classes/SetoidDec.v index f4220e3aa1..435dacbd4c 100644 --- a/theories/Classes/SetoidDec.v +++ b/theories/Classes/SetoidDec.v @@ -42,7 +42,7 @@ Class EqDec `(S : Setoid A) := take precedence of [==] defined in the type scope, hence we can have both at the same time. *) -Notation " x == y " := (equiv_dec (x :>) (y :>)) (no associativity, at level 70). +Notation " x == y " := (equiv_dec x y) (no associativity, at level 70). Definition swap_sumbool {A B} (x : { A } + { B }) : { B } + { A } := match x with |
