aboutsummaryrefslogtreecommitdiffhomepage
path: root/plugins/ssr/ssrview.mli
blob: 6fd906ff4f037f6b739ff257e8b3bccc4749d706 (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
36
(************************************************************************)
(*  v      *   The Coq Proof Assistant  /  The Coq Development Team     *)
(* <O___,, *   INRIA - CNRS - LIX - LRI - PPS - Copyright 1999-2017     *)
(*   \VV/  **************************************************************)
(*    //   *      This file is distributed under the terms of the       *)
(*         *       GNU Lesser General Public License Version 2.1        *)
(************************************************************************)

(* This file is (C) Copyright 2006-2015 Microsoft Corporation and Inria. *)

open Ssrast
open Ssrcommon

val viewtab : Glob_term.glob_constr list array
val add_view_hints : Glob_term.glob_constr list -> int -> unit
val glob_view_hints : Constrexpr.constr_expr list -> Glob_term.glob_constr list

val pfa_with_view :
           ist ->
           ?next:ssripats ref ->
           bool * ssrterm list ->
           EConstr.t ->
           EConstr.t ->
           (EConstr.t -> EConstr.t -> tac_ctx tac_a) ->
           ssrhyps ->
   (goal * tac_ctx) sigma -> EConstr.types * EConstr.t * (goal * tac_ctx) list sigma

val pf_with_view_linear :
           ist ->
           goal sigma ->
           bool * ssrterm list ->
           EConstr.t ->
           EConstr.t ->
           EConstr.types * EConstr.t * goal sigma