aboutsummaryrefslogtreecommitdiffhomepage
path: root/proofs/logic.mli
blob: 4d1c2de9791687216d83a264d696601fb1715994 (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
37
38
39
40
41
42

(* $Id$ *)

(*i*)
open Names
open Term
open Sign
open Evd
open Environ
open Proof_trees
(*i*)

(* The primitive refiner. *)

val prim_refiner : prim_rule -> 'a evar_map -> goal -> goal list

val prim_extractor : 
  ((typed_type, constr) sign -> proof_tree -> constr) -> 
    (typed_type, constr) sign -> proof_tree -> constr

val extract_constr : constr assumptions -> constr -> constr


(*s Refiner errors. *)

type refiner_error =
  | BadType of constr * constr * constr
  | OccurMeta of constr
  | CannotApply of constr * constr
  | CannotUnify of constr * constr
  | CannotGeneralize of typed_type signature * constr
  | NotWellTyped of constr
  | BadTacticArgs of string * tactic_arg list

exception RefinerError of refiner_error

val error_cannot_unify : path_kind -> constr * constr -> 'a


(*s Pretty-printer. *)

val pr_prim_rule   : prim_rule -> Pp.std_ppcmds