diff options
| author | Jasper Hugunin | 2021-01-08 12:42:47 -0800 |
|---|---|---|
| committer | Jasper Hugunin | 2021-01-08 12:42:47 -0800 |
| commit | 7dd5f0cc776f0a79b3852cd1ed30fa0edab17a73 (patch) | |
| tree | db4b78dd98ca9e80e98003911014acc0ff57f0fe | |
| parent | 76cbd4afbeb13d97852e97e805c0e1890eae1d6c (diff) | |
Modify Classes/EquivDec.v to compile with -mangle-names
| -rw-r--r-- | theories/Classes/EquivDec.v | 7 |
1 files changed, 5 insertions, 2 deletions
diff --git a/theories/Classes/EquivDec.v b/theories/Classes/EquivDec.v index 6978fa1ddf..a1a4da6f37 100644 --- a/theories/Classes/EquivDec.v +++ b/theories/Classes/EquivDec.v @@ -87,7 +87,7 @@ Program Instance unit_eqdec : EqDec unit eq := fun x y => in_left. Next Obligation. Proof. - destruct x ; destruct y. + do 2 match goal with [ x : () |- _ ] => destruct x end. reflexivity. Qed. @@ -142,7 +142,10 @@ Program Instance list_eqdec `(eqa : EqDec A eq) : EqDec (list A) eq := | _, _ => in_right end }. - Next Obligation. destruct y ; unfold not in *; eauto. Defined. + Next Obligation. + match goal with y : list _ |- _ => destruct y end ; + unfold not in *; eauto. + Defined. Solve Obligations with unfold equiv, complement in * ; program_simpl ; intuition (discriminate || eauto). |
