aboutsummaryrefslogtreecommitdiff
path: root/mathcomp/ssreflect/choice.v
diff options
context:
space:
mode:
authorCyril Cohen2020-11-20 02:31:40 +0100
committerCyril Cohen2020-11-20 20:50:44 +0100
commitc55acd1fefa970cc4ed3a8a53b05fd77008a7cdf (patch)
tree864b98bd44a865c6155e96746a4c837061a51888 /mathcomp/ssreflect/choice.v
parentfd0d84084738decce3fb6557cf82dc10d030daa8 (diff)
Tuning simplifications using Arguments simpl nomatch
Diffstat (limited to 'mathcomp/ssreflect/choice.v')
-rw-r--r--mathcomp/ssreflect/choice.v1
1 files changed, 1 insertions, 0 deletions
diff --git a/mathcomp/ssreflect/choice.v b/mathcomp/ssreflect/choice.v
index a68ec41..81b83dc 100644
--- a/mathcomp/ssreflect/choice.v
+++ b/mathcomp/ssreflect/choice.v
@@ -76,6 +76,7 @@ Fixpoint decode_rec (v q r : nat) {struct q} :=
| q'.+1, 1 => [rec v.+1, q', q']
| q'.+1, r'.+2 => [rec v, q', r']
end where "[ 'rec' v , q , r ]" := (decode_rec v q r).
+Arguments decode_rec : simpl nomatch.
Definition decode n := if n is 0 then [::] else [rec 0, n.-1, n.-1].