aboutsummaryrefslogtreecommitdiffhomepage
path: root/contrib/subtac/Utils.v
diff options
context:
space:
mode:
authorGravatar msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7>2007-02-07 20:12:34 +0000
committerGravatar msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7>2007-02-07 20:12:34 +0000
commit13223ba6649dfd7501a34a700abc09c2e7169636 (patch)
tree626096576a69f19470ee2d2682373cc7469f99a9 /contrib/subtac/Utils.v
parentddbfb9299340f069a26fc6218e82031a8a99d056 (diff)
Add tactics for induction on subterms.
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@9623 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'contrib/subtac/Utils.v')
-rw-r--r--contrib/subtac/Utils.v4
1 files changed, 4 insertions, 0 deletions
diff --git a/contrib/subtac/Utils.v b/contrib/subtac/Utils.v
index 569c52e89..fc002a01b 100644
--- a/contrib/subtac/Utils.v
+++ b/contrib/subtac/Utils.v
@@ -4,6 +4,8 @@ Notation "'fun' { x : A | P } => Q" :=
(fun x:{x:A|P} => Q)
(at level 200, x ident, right associativity).
+Notation " {{ x }} " := (tt : { y : unit | x }).
+
Notation "( x & ? )" := (@exist _ _ x _) : core_scope.
Notation " ! " := (False_rect _ _).
@@ -82,6 +84,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" [ "" ].