aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/success/intros.v
diff options
context:
space:
mode:
Diffstat (limited to 'test-suite/success/intros.v')
-rw-r--r--test-suite/success/intros.v14
1 files changed, 14 insertions, 0 deletions
diff --git a/test-suite/success/intros.v b/test-suite/success/intros.v
index 11156aa0e..69d66f100 100644
--- a/test-suite/success/intros.v
+++ b/test-suite/success/intros.v
@@ -84,3 +84,17 @@ Qed.
Goal forall x : nat, True.
intros y%(fun x => x).
Abort.
+
+(* Fixing a bug in the order of side conditions of a "->" step *)
+
+Goal (True -> 1=0) -> 1=1.
+intros ->.
+- reflexivity.
+- exact I.
+Qed.
+
+Goal forall x, (True -> x=0) -> 0=x.
+intros x ->.
+- reflexivity.
+- exact I.
+Qed.