aboutsummaryrefslogtreecommitdiffhomepage
path: root/pretyping/recordops.mli
blob: 7402f74c9a5cc918c3fa6ff8d67c607bd8488e1a (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
43
44
45
46
47
48
49
50
51
52
53
(************************************************************************)
(*  v      *   The Coq Proof Assistant  /  The Coq Development Team     *)
(* <O___,, * CNRS-Ecole Polytechnique-INRIA Futurs-Universite Paris Sud *)
(*   \VV/  **************************************************************)
(*    //   *      This file is distributed under the terms of the       *)
(*         *       GNU Lesser General Public License Version 2.1        *)
(************************************************************************)

(*i $Id$ i*)

(*i*)
open Names
open Nametab
open Term
open Libnames
open Classops
open Libobject
open Library
(*i*)

type struc_typ = {
  s_CONST : identifier; 
  s_PARAM : int;
  s_PROJ : constant option list }

val add_new_struc : 
  inductive * identifier * int * constant option list -> unit

(* [find_structure isp] returns the infos associated to inductive path
   [isp] if it corresponds to a structure, otherwise fails with [Not_found] *)
val find_structure : inductive -> struc_typ

(* raise [Not_found] if not a projection *)
val find_projection_nparams : global_reference -> int

type obj_typ = {
  o_DEF : constr;
  o_TABS : constr list; (* dans l'ordre *)
  o_TPARAMS : constr list; (* dans l'ordre *)
  o_TCOMPS : constr list } (* dans l'ordre *)
               
val canonical_structure_info : 
  (global_reference * global_reference) -> obj_typ
val add_canonical_structure : 
  constant * ((global_reference * global_reference) * obj_typ) list -> unit

val inStruc : inductive * struc_typ -> obj
val outStruc : obj -> inductive * struc_typ

val outCanonicalStructure : obj -> constant

val canonical_structures : unit -> 
  ((global_reference * global_reference) * obj_typ) list