diff options
author | letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7> | 2003-11-12 16:46:06 +0000 |
---|---|---|
committer | letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7> | 2003-11-12 16:46:06 +0000 |
commit | f52d396b1c1499cb12531d89e77341326192b53d (patch) | |
tree | 2e6530ffaae97d8c790d1de886c3889586c02bfd /doc/Extraction.tex | |
parent | 06807ca5dab501303aa63571838813ab388d7097 (diff) |
En fait les Import des Require sont de nouveau utiles
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@8353 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'doc/Extraction.tex')
-rwxr-xr-x | doc/Extraction.tex | 12 |
1 files changed, 6 insertions, 6 deletions
diff --git a/doc/Extraction.tex b/doc/Extraction.tex index 0ad4410b1..629b84530 100755 --- a/doc/Extraction.tex +++ b/doc/Extraction.tex @@ -369,7 +369,7 @@ We can now extract this program to \ocaml: Reset Initial. \end{coq_eval} \begin{coq_example} -Require Euclid. +Require Import Euclid. Extraction Inline Wf_nat.gt_wf_rec Wf_nat.lt_wf_rec. Recursive Extraction eucl_dev. \end{coq_example} @@ -421,13 +421,13 @@ treesort}, whose type is shown below: \begin{coq_eval} Reset Initial. -Require Relation_Definitions. -Require List. -Require Sorting. -Require Permutation. +Require Import Relation_Definitions. +Require Import List. +Require Import Sorting. +Require Import Permutation. \end{coq_eval} \begin{coq_example} -Require Heap. +Require Import Heap. Check treesort. \end{coq_example} |