summaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/38.v
diff options
context:
space:
mode:
authorGravatar Benjamin Barenblat <bbaren@debian.org>2018-12-29 14:31:27 -0500
committerGravatar Benjamin Barenblat <bbaren@debian.org>2018-12-29 14:31:27 -0500
commit9043add656177eeac1491a73d2f3ab92bec0013c (patch)
tree2b0092c84bfbf718eca10c81f60b2640dc8cab05 /test-suite/bugs/closed/38.v
parenta4c7f8bd98be2a200489325ff7c5061cf80ab4f3 (diff)
Imported Upstream version 8.8.2upstream/8.8.2
Diffstat (limited to 'test-suite/bugs/closed/38.v')
-rw-r--r--test-suite/bugs/closed/38.v22
1 files changed, 0 insertions, 22 deletions
diff --git a/test-suite/bugs/closed/38.v b/test-suite/bugs/closed/38.v
deleted file mode 100644
index 4fc8d7c9..00000000
--- a/test-suite/bugs/closed/38.v
+++ /dev/null
@@ -1,22 +0,0 @@
-Require Import Setoid.
-
-Variable A : Set.
-
-Inductive liste : Set :=
-| vide : liste
-| c : A -> liste -> liste.
-
-Inductive e : A -> liste -> Prop :=
-| ec : forall (x : A) (l : liste), e x (c x l)
-| ee : forall (x y : A) (l : liste), e x l -> e x (c y l).
-
-Definition same := fun (l m : liste) => forall (x : A), e x l <-> e x m.
-
-Definition same_refl (x:liste) : (same x x).
- unfold same; split; intros; trivial.
-Save.
-
-Goal forall (x:liste), (same x x).
- intro.
- apply (same_refl x).
-Qed.