diff options
author | herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7> | 2003-10-21 08:40:35 +0000 |
---|---|---|
committer | herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7> | 2003-10-21 08:40:35 +0000 |
commit | a45a6ce02092bdf9ca906dd57a515030e3b17422 (patch) | |
tree | 867ca66a59795873425e34cd456d325905bcaf26 /theories/Init | |
parent | 327c9115cf88d919d8f6b17904764c4147116604 (diff) |
Maintenant avant Datatypes
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@4681 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Init')
-rwxr-xr-x | theories/Init/Logic.v | 1 |
1 files changed, 0 insertions, 1 deletions
diff --git a/theories/Init/Logic.v b/theories/Init/Logic.v index 683058420..680b1e20e 100755 --- a/theories/Init/Logic.v +++ b/theories/Init/Logic.v @@ -12,7 +12,6 @@ Set Implicit Arguments. V7only [Unset Implicit Arguments.]. Require Notations. -Require Datatypes. (** [True] is the always true proposition *) Inductive True : Prop := I : True. |