diff options
author | msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7> | 2007-07-02 12:38:33 +0000 |
---|---|---|
committer | msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7> | 2007-07-02 12:38:33 +0000 |
commit | 7347565231d027255f4d24d7daff06cc07c5e5c9 (patch) | |
tree | ec0173673ae601863f70d7a1443cd2bb367c573e /contrib/subtac/Utils.v | |
parent | 0bd7be45957ae556074aa5a12bdc66df1726065a (diff) |
Better handling of aliases, add command to solve a particular obligation.
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@9929 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'contrib/subtac/Utils.v')
-rw-r--r-- | contrib/subtac/Utils.v | 6 |
1 files changed, 2 insertions, 4 deletions
diff --git a/contrib/subtac/Utils.v b/contrib/subtac/Utils.v index a83a321de..1d19dbd19 100644 --- a/contrib/subtac/Utils.v +++ b/contrib/subtac/Utils.v @@ -42,10 +42,8 @@ Extraction Inline proj1_sig. Extract Inductive unit => "unit" [ "()" ]. Extract Inductive bool => "bool" [ "true" "false" ]. Extract Inductive sumbool => "bool" [ "true" "false" ]. -Axiom pair : Type -> Type -> Type. -Extract Constant pair "'a" "'b" => " 'a * 'b ". -Extract Inductive prod => "pair" [ "" ]. -Extract Inductive sigT => "pair" [ "" ]. +(* Extract Inductive prod "'a" "'b" => " 'a * 'b " [ "(,)" ]. *) +(* Extract Inductive sigT => "prod" [ "" ]. *) Require Export ProofIrrelevance. Require Export Coq.subtac.Heq. |