Skip to content

Commit

Permalink
Make Permutation_cons and _app' #[export]
Browse files Browse the repository at this point in the history
Fix coq#15596 (we still get a slowdown on Require Import)
Maybe we should use Hint Extern or just don't declare these Proper
instances instead.
  • Loading branch information
SkySkimmer committed Feb 3, 2022
1 parent 7d14801 commit ecdb3db
Showing 1 changed file with 2 additions and 2 deletions.
4 changes: 2 additions & 2 deletions theories/Sorting/Permutation.v
Expand Up @@ -106,7 +106,7 @@ Proof.
now apply IHHP; rewrite <- app_assoc.
Qed.

#[global]
#[export]
Instance Permutation_cons A :
Proper (Logic.eq ==> @Permutation A ==> @Permutation A) (@cons A).
Proof.
Expand Down Expand Up @@ -161,7 +161,7 @@ Proof.
apply Permutation_app_tail; assumption.
Qed.

Global Instance Permutation_app' :
#[export] Instance Permutation_app' :
Proper (@Permutation A ==> @Permutation A ==> @Permutation A) (@app A).
Proof.
repeat intro; now apply Permutation_app.
Expand Down

0 comments on commit ecdb3db

Please sign in to comment.