blob: 32ae18a79e9477975de48dd137d004d6ff2fd447 (
plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
16
17
18
19
20
21
22
23
24
25
26
27
28
29
30
31
32
33
34
35
|
(************************************************************************)
(* * The Coq Proof Assistant / The Coq Development Team *)
(* v * Copyright INRIA, CNRS and contributors *)
(* <O___,, * (see version control and CREDITS file for authors & dates) *)
(* \VV/ **************************************************************)
(* // * This file is distributed under the terms of the *)
(* * GNU Lesser General Public License Version 2.1 *)
(* * (see LICENSE file for the text of the license) *)
(************************************************************************)
open Names
open EConstr
(** This file extends Matching with the main logic for Ltac2 match goal. *)
type context = EConstr.t
type match_pattern =
| MatchPattern of Pattern.constr_pattern
| MatchContext of Pattern.constr_pattern
(** TODO: handle definitions *)
type match_context_hyps = match_pattern
type match_rule = match_context_hyps list * match_pattern
val match_goal:
Environ.env ->
Evd.evar_map ->
constr ->
rev:bool ->
match_rule ->
((Id.t * context option) list * (* List of hypotheses matching: name + context *)
context option * (* Context for conclusion *)
Ltac_pretype.patvar_map (* Pattern variable substitution *)) Proofview.tactic
|