products/sources/formale Sprachen/Coq/test-suite/output image not shown  

Quellcode-Bibliothek

© Kompilation durch diese Firma

[Weder Korrektheit noch Funktionsfähigkeit der Software werden zugesichert.]

Datei: ShowExtraction.v   Sprache: Unknown


Require Extraction.
Require Import List.

Section Test.
Variable A : Type.
Variable decA : forall (x y:A), {x=y}+{x<>y}.

(** Should fail when no proofs are started *)
Fail Show Extraction.

Lemma decListA : forall (xs ys : list A), {xs=ys}+{xs<>ys}.
Proof.
Show Extraction.
fix decListA 1.
destruct xs as [|x xs], ys as [|y ys].
Show Extraction.
now left.
now right.
now right.
- Show Extraction.
  destruct (decA x y).
  + destruct (decListA xs ys).
    * leftnow f_equal.
    * Show Extraction.
      right. congruence.
  + right. congruence.
Show Extraction.
Defined.

End Test.

[ Dauer der Verarbeitung: 0.1 Sekunden  (vorverarbeitet)  ]