(** Bug 4709 https://coq.inria.fr/bug/4709
Extraction wasn't reducing primitive projections in types. *)
Require Extraction.
Set Primitive Projections.
Record t := Foo { foo : Type }.
Definition ty := foo (Foo nat).
(* Without proper reduction of primitive projections in
[extract_type], the type [ty] was extracted as [Tunknown].
Let's check it isn't the case anymore. *)
Parameter check : nat.
Extract Constant check => "(O:ty)".
Extraction TestCompile ty check.
¤ Dauer der Verarbeitung: 0.16 Sekunden
(vorverarbeitet)
¤
|
Haftungshinweis
Die Informationen auf dieser Webseite wurden
nach bestem Wissen sorgfältig zusammengestellt. Es wird jedoch weder Vollständigkeit, noch Richtigkeit,
noch Qualität der bereit gestellten Informationen zugesichert.
Bemerkung:
Die farbliche Syntaxdarstellung ist noch experimentell.
|