diff options
author | filliatr <filliatr@85f007b7-540e-0410-9357-904b9bb8a0f7> | 2007-02-14 08:09:05 +0000 |
---|---|---|
committer | filliatr <filliatr@85f007b7-540e-0410-9357-904b9bb8a0f7> | 2007-02-14 08:09:05 +0000 |
commit | 2e1e80b173846c8ed7ac94ce5f533ffc6cd6c8bd (patch) | |
tree | 4d8bd342c8fbb1cac7bb05ef47ea81ff13acc605 /contrib/dp/tests.v | |
parent | 3786c49aadcd609151c44b2458c00cf612b807bb (diff) |
encodage des types
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@9646 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'contrib/dp/tests.v')
-rw-r--r-- | contrib/dp/tests.v | 5 |
1 files changed, 3 insertions, 2 deletions
diff --git a/contrib/dp/tests.v b/contrib/dp/tests.v index 984d66c8f..b32c45e74 100644 --- a/contrib/dp/tests.v +++ b/contrib/dp/tests.v @@ -4,6 +4,9 @@ Require Import Classical. Require Export zenon. +Dp_debug. +Dp_timeout 3. + (* First example with the 0 and the equality translated *) Goal 0 = 0. @@ -39,8 +42,6 @@ Goal ((((A -> C) -> A) -> A) -> C) -> C. zenon. Qed. -Dp_debug. - (* Arithmetic *) Open Scope Z_scope. |