aboutsummaryrefslogtreecommitdiff
path: root/mathcomp/discrete/path.v
diff options
context:
space:
mode:
authorCyril Cohen2015-04-03 17:22:31 +0200
committerCyril Cohen2015-04-03 17:22:31 +0200
commit9fa572c64085bc020edee574a694fe0805fefdfa (patch)
tree14da7c2ee40df06402679f146c450106a0fab03b /mathcomp/discrete/path.v
parent9859058e3dff7c4ba8153b5e5adb10043faa5807 (diff)
prepared discrete for compilation in v8.5
Diffstat (limited to 'mathcomp/discrete/path.v')
-rw-r--r--mathcomp/discrete/path.v1
1 files changed, 1 insertions, 0 deletions
diff --git a/mathcomp/discrete/path.v b/mathcomp/discrete/path.v
index 804e673..85746a4 100644
--- a/mathcomp/discrete/path.v
+++ b/mathcomp/discrete/path.v
@@ -1,4 +1,5 @@
(* (c) Copyright Microsoft Corporation and Inria. All rights reserved. *)
+(*v8.5 From mathcomp.ssreflect *)
Require Import ssreflect ssrfun ssrbool eqtype ssrnat seq.
(******************************************************************************)