aboutsummaryrefslogtreecommitdiffhomepage
path: root/contrib/extraction/test_extraction.v
diff options
context:
space:
mode:
authorGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2002-07-16 12:45:39 +0000
committerGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2002-07-16 12:45:39 +0000
commitf71117475f0ae994c107c7b9e7ea48c9a7a6514f (patch)
tree70be735b5a47ba3a272def311e2b66fea3744993 /contrib/extraction/test_extraction.v
parentea41376804c30a583377c0ca45ad8e1b378838df (diff)
Gros Remaniement Extraction:
* extraction.ml + modulaire (cf extract_type) et + proche theorie (cf feu extract_app) * table.ml filtre les Extract Constant vers types ou terms * extract_env.ml refuse maintenant les Extraction constr. git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@2886 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'contrib/extraction/test_extraction.v')
-rw-r--r--contrib/extraction/test_extraction.v9
1 files changed, 9 insertions, 0 deletions
diff --git a/contrib/extraction/test_extraction.v b/contrib/extraction/test_extraction.v
index ef7d80e0c..44aeff317 100644
--- a/contrib/extraction/test_extraction.v
+++ b/contrib/extraction/test_extraction.v
@@ -388,3 +388,12 @@ let oups h0 = match h0 with
Extraction (sigT Set [a:Set](option a)).
(* (unit, Obj.t option) sigT *)
+
+(* Coq term non strongly-normalizable after extraction *)
+
+Require Gt.
+Definition loop :=
+ [Ax:(Acc nat gt O)]
+ (Fix F {F [a:nat;b:(Acc nat gt a)] : nat :=
+ (F (S a) (Acc_inv nat gt a b (S a) (gt_Sn_n a)))}
+ O Ax). \ No newline at end of file