aboutsummaryrefslogtreecommitdiffhomepage
path: root/contrib/subtac/Utils.v
diff options
context:
space:
mode:
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" [ "" ].