aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Init/Wf.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-09-23 11:23:14 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-09-23 11:23:14 +0000
commit58b3bc4b3151bc5f8b81fbc7a1943f99b081f80e (patch)
tree32269fe01cb1488a1d6ab4e0a9d0ec64efb3deee /theories/Init/Wf.v
parent4d7184fe2f570f123eef72c88d6d3f082617bd2a (diff)
Fusion des fichiers de syntaxe de Init avec les fichiers de définition; TypeSyntax inutile
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@4461 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Init/Wf.v')
-rwxr-xr-xtheories/Init/Wf.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/Init/Wf.v b/theories/Init/Wf.v
index 93111571f..fbc71a3ea 100755
--- a/theories/Init/Wf.v
+++ b/theories/Init/Wf.v
@@ -17,8 +17,8 @@ V7only [Unset Implicit Arguments.].
from a well-founded ordering on a given set *)
+Require Notations.
Require Logic.
-Require LogicSyntax.
Require Datatypes.
(** Well-founded induction principle on Prop *)