aboutsummaryrefslogtreecommitdiff
path: root/mathcomp/ssreflect/path.v
diff options
context:
space:
mode:
authorCyril Cohen2019-04-26 14:14:15 +0200
committerCyril Cohen2019-04-26 15:08:48 +0200
commit22c182b681c2852afa13efc2bc1d6d083646f061 (patch)
tree240ce34774221645650404da1337e94c5e3f63b3 /mathcomp/ssreflect/path.v
parentdec1f90d13c44016ea53da360e9692fd768bc24b (diff)
Cleaning Require and Require Imports
Diffstat (limited to 'mathcomp/ssreflect/path.v')
-rw-r--r--mathcomp/ssreflect/path.v4
1 files changed, 1 insertions, 3 deletions
diff --git a/mathcomp/ssreflect/path.v b/mathcomp/ssreflect/path.v
index b6bc4ed..4d0d208 100644
--- a/mathcomp/ssreflect/path.v
+++ b/mathcomp/ssreflect/path.v
@@ -1,8 +1,6 @@
(* (c) Copyright 2006-2016 Microsoft Corporation and Inria. *)
(* Distributed under the terms of CeCILL-B. *)
-Require Import mathcomp.ssreflect.ssreflect.
-From mathcomp
-Require Import ssrfun ssrbool eqtype ssrnat seq.
+From mathcomp Require Import ssreflect ssrfun ssrbool eqtype ssrnat seq.
(******************************************************************************)
(* The basic theory of paths over an eqType; this file is essentially a *)