aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/success
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2009-12-29 21:22:21 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2009-12-29 21:22:21 +0000
commit77d86619f5f557de52a391f6811bacd73c01580b (patch)
treeb4a761531c326034b257ad6503a94dec6d2c7485 /test-suite/success
parent5fabc3437c152522b6b4d86d3deb134e5de228ab (diff)
Renouncing to have the option "Automatic Introduction" on by default.
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@12613 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'test-suite/success')
-rw-r--r--test-suite/success/Fixpoint.v2
1 files changed, 2 insertions, 0 deletions
diff --git a/test-suite/success/Fixpoint.v b/test-suite/success/Fixpoint.v
index fcf8d8d4a..3a4f88993 100644
--- a/test-suite/success/Fixpoint.v
+++ b/test-suite/success/Fixpoint.v
@@ -50,6 +50,8 @@ End folding.
(* Check definition by tactics *)
+Set Automatic Introduction.
+
Inductive even : nat -> Type :=
| even_O : even 0
| even_S : forall n, odd n -> even (S n)