aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Logic
diff options
context:
space:
mode:
authorGravatar Pierre Boutillier <pierre.boutillier@ens-lyon.org>2014-02-20 17:39:15 +0100
committerGravatar Pierre Boutillier <pierre.boutillier@ens-lyon.org>2014-02-24 14:07:07 +0100
commit26c390aae1275f02892412f121360668ad98a660 (patch)
tree4fd13daac049adc7b618d115766fb025f9637ec0 /theories/Logic
parent80410d825befa1890c872596cf77378a437cee73 (diff)
fixup complement Fin
Diffstat (limited to 'theories/Logic')
-rw-r--r--theories/Logic/FinFun.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/Logic/FinFun.v b/theories/Logic/FinFun.v
index f070a6889..2f72f16de 100644
--- a/theories/Logic/FinFun.v
+++ b/theories/Logic/FinFun.v
@@ -245,7 +245,7 @@ Notation n2f := Fin.of_nat_lt.
Definition f2n {n} (x:Fin.t n) := proj1_sig (Fin.to_nat x).
Definition f2n_ok n (x:Fin.t n) : f2n x < n := proj2_sig (Fin.to_nat x).
Definition n2f_f2n : forall n x, n2f (f2n_ok x) = x := @Fin.of_nat_to_nat_inv.
-Definition f2n_n2f : forall x n h, f2n (n2f h) = x := @Fin.to_nat_of_nat.
+Definition f2n_n2f x n h : f2n (n2f h) = x := f_equal (@proj1_sig _ _) (@Fin.to_nat_of_nat x n h).
Definition n2f_ext : forall x n h h', n2f h = n2f h' := @Fin.of_nat_ext.
Definition f2n_inj : forall n x y, f2n x = f2n y -> x = y := @Fin.to_nat_inj.