aboutsummaryrefslogtreecommitdiffhomepage
path: root/tactics
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2000-09-10 21:22:57 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2000-09-10 21:22:57 +0000
commitc039e4e618d7da96909d42995eb21074945a3624 (patch)
treea58d5f6393afb1e66b1ee9e73f8bd492acc534be /tactics
parente72024e2292a50684b7f280d6efb8fee090e2dbf (diff)
Correction pour make doc
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@594 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'tactics')
-rw-r--r--tactics/auto.ml2
-rw-r--r--tactics/btermdn.mli2
-rw-r--r--tactics/dhyp.ml2
-rw-r--r--tactics/eauto.ml2
-rw-r--r--tactics/elim.ml2
-rw-r--r--tactics/equality.ml2
-rw-r--r--tactics/hipattern.ml2
-rw-r--r--tactics/inv.ml2
-rw-r--r--tactics/leminv.ml2
-rw-r--r--tactics/nbtermdn.ml2
-rw-r--r--tactics/nbtermdn.mli2
-rw-r--r--tactics/refine.ml2
-rw-r--r--tactics/tacticals.ml2
-rw-r--r--tactics/tactics.ml2
-rw-r--r--tactics/tauto.ml2
-rw-r--r--tactics/termdn.ml2
-rw-r--r--tactics/termdn.mli2
-rw-r--r--tactics/wcclausenv.ml2
18 files changed, 18 insertions, 18 deletions
diff --git a/tactics/auto.ml b/tactics/auto.ml
index e5dfff04c..acf0b6cc6 100644
--- a/tactics/auto.ml
+++ b/tactics/auto.ml
@@ -4,7 +4,7 @@
open Pp
open Util
open Names
-(*i open Generic i*)
+(* open Generic *)
open Term
open Sign
open Inductive
diff --git a/tactics/btermdn.mli b/tactics/btermdn.mli
index aeb3f306c..ca1d0831a 100644
--- a/tactics/btermdn.mli
+++ b/tactics/btermdn.mli
@@ -2,7 +2,7 @@
(* $Id$ *)
(*i*)
-(*i open Generic i*)
+(* open Generic *)
open Term
open Pattern
(*i*)
diff --git a/tactics/dhyp.ml b/tactics/dhyp.ml
index 4190cb17d..7e3ac13b2 100644
--- a/tactics/dhyp.ml
+++ b/tactics/dhyp.ml
@@ -107,7 +107,7 @@ Qed.
open Pp
open Util
open Names
-(*i open Generic i*)
+(* open Generic *)
open Term
open Environ
open Reduction
diff --git a/tactics/eauto.ml b/tactics/eauto.ml
index 6eab9ae08..09d8885d8 100644
--- a/tactics/eauto.ml
+++ b/tactics/eauto.ml
@@ -4,7 +4,7 @@
open Pp
open Util
open Names
-(*i open Generic i*)
+(* open Generic *)
open Term
open Sign
open Reduction
diff --git a/tactics/elim.ml b/tactics/elim.ml
index 0fbfcae9a..2cfcd8559 100644
--- a/tactics/elim.ml
+++ b/tactics/elim.ml
@@ -4,7 +4,7 @@
open Pp
open Util
open Names
-(*i open Generic i*)
+(* open Generic *)
open Term
open Reduction
open Inductive
diff --git a/tactics/equality.ml b/tactics/equality.ml
index f32562182..bec81d44a 100644
--- a/tactics/equality.ml
+++ b/tactics/equality.ml
@@ -5,7 +5,7 @@ open Pp
open Util
open Names
open Univ
-(*i open Generic i*)
+(* open Generic *)
open Term
open Inductive
open Environ
diff --git a/tactics/hipattern.ml b/tactics/hipattern.ml
index fd54744fe..cc88fbcd7 100644
--- a/tactics/hipattern.ml
+++ b/tactics/hipattern.ml
@@ -4,7 +4,7 @@
open Pp
open Util
open Names
-(*i open Generic i*)
+(* open Generic *)
open Term
open Reduction
open Inductive
diff --git a/tactics/inv.ml b/tactics/inv.ml
index 82863269b..0a09c441b 100644
--- a/tactics/inv.ml
+++ b/tactics/inv.ml
@@ -4,7 +4,7 @@
open Pp
open Util
open Names
-(*i open Generic i*)
+(* open Generic *)
open Term
open Global
open Sign
diff --git a/tactics/leminv.ml b/tactics/leminv.ml
index 57baf0b15..c5bf51771 100644
--- a/tactics/leminv.ml
+++ b/tactics/leminv.ml
@@ -4,7 +4,7 @@
open Pp
open Util
open Names
-(*i open Generic i*)
+(* open Generic *)
open Term
open Sign
open Evd
diff --git a/tactics/nbtermdn.ml b/tactics/nbtermdn.ml
index ae0f5a6c9..d5d657365 100644
--- a/tactics/nbtermdn.ml
+++ b/tactics/nbtermdn.ml
@@ -3,7 +3,7 @@
open Util
open Names
-(*i open Generic i*)
+(* open Generic *)
open Term
open Libobject
open Library
diff --git a/tactics/nbtermdn.mli b/tactics/nbtermdn.mli
index f68fc89e7..4cbf696c4 100644
--- a/tactics/nbtermdn.mli
+++ b/tactics/nbtermdn.mli
@@ -2,7 +2,7 @@
(* $Id$ *)
(*i*)
-(*i open Generic i*)
+(* open Generic *)
open Term
open Pattern
(*i*)
diff --git a/tactics/refine.ml b/tactics/refine.ml
index f5a95d59c..08105aa9f 100644
--- a/tactics/refine.ml
+++ b/tactics/refine.ml
@@ -42,7 +42,7 @@
open Pp
open Util
open Names
-(*i open Generic i*)
+(* open Generic *)
open Term
open Tacmach
open Sign
diff --git a/tactics/tacticals.ml b/tactics/tacticals.ml
index b77ac413c..d5ee7f965 100644
--- a/tactics/tacticals.ml
+++ b/tactics/tacticals.ml
@@ -4,7 +4,7 @@
open Pp
open Util
open Names
-(*i open Generic i*)
+(* open Generic *)
open Term
open Sign
open Declarations
diff --git a/tactics/tactics.ml b/tactics/tactics.ml
index 4312071b4..a8693a70b 100644
--- a/tactics/tactics.ml
+++ b/tactics/tactics.ml
@@ -6,7 +6,7 @@ open Util
open Stamps
open Names
open Sign
-(*i open Generic i*)
+(* open Generic *)
open Term
open Inductive
open Reduction
diff --git a/tactics/tauto.ml b/tactics/tauto.ml
index 416e81cd2..7c00a6b1d 100644
--- a/tactics/tauto.ml
+++ b/tactics/tauto.ml
@@ -6,7 +6,7 @@
open Pp
open Util
open Names
-(*i open Generic i*)
+(* open Generic *)
open Term
open Sign
open Environ
diff --git a/tactics/termdn.ml b/tactics/termdn.ml
index 9cdb34ab2..920e6ba31 100644
--- a/tactics/termdn.ml
+++ b/tactics/termdn.ml
@@ -2,7 +2,7 @@
(* $Id$ *)
open Util
-(*i open Generic i*)
+(* open Generic *)
open Names
open Term
open Pattern
diff --git a/tactics/termdn.mli b/tactics/termdn.mli
index 107026ef6..02415bc3c 100644
--- a/tactics/termdn.mli
+++ b/tactics/termdn.mli
@@ -2,7 +2,7 @@
(* $Id$ *)
(*i*)
-(*i open Generic i*)
+(* open Generic *)
open Term
open Pattern
(*i*)
diff --git a/tactics/wcclausenv.ml b/tactics/wcclausenv.ml
index 25c63e536..4f071980e 100644
--- a/tactics/wcclausenv.ml
+++ b/tactics/wcclausenv.ml
@@ -4,7 +4,7 @@
open Pp
open Util
open Names
-(*i open Generic i*)
+(* open Generic *)
open Term
open Sign
open Reduction