aboutsummaryrefslogtreecommitdiffhomepage
path: root/pretyping/retyping.ml
blob: 51f7e66e302a4c581db01b0cad94aa7562ce0b0d (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
54
55
56
57
58
59
60
61
62
63
64
65
66
67
68
69
70
71
72
73
74
75
76
77
78
79
80
81
82
83
84
85
86
87
88
89
90
91
92
93
94
95
96

(* $Id$ *)

open Util
open Term
open Inductive
open Names
open Generic
open Reduction
open Environ
open Typeops

type metamap = (int * constr) list

let outsort env sigma t =
  match whd_betadeltaiota env sigma t with
      DOP0(Sort s) -> s
    | _ -> anomaly "outsort: Not a sort"

let rec subst_type env sigma typ = function
    [] -> typ
  | h::rest ->
      match whd_betadeltaiota env sigma typ with
          DOP2(Prod,c1,DLAM(_,c2)) -> subst_type env sigma (subst1 h c2) rest
        | _ -> anomaly "Non-functional construction"

(* Si ft est le type d'un terme f, lequel est appliqué à args, *)
(* [sort_of_atomic_ty] calcule ft[args] qui doit être une sorte *)
(* On suit une méthode paresseuse, en espèrant que ft est une arité *)
(* et sinon on substitue *)

let sort_of_atomic_type env sigma ft args =
  let rec concl_of_arity ar =
    match whd_betadeltaiota env sigma ar with
      | DOP2 (Prod, _, DLAM (_, b)) -> concl_of_arity b
      | DOP0 (Sort s) -> s
      | _ -> outsort env sigma (subst_type env sigma ft args)
  in concl_of_arity ft

let typeur sigma metamap =
let rec type_of env cstr=
  match kind_of_term cstr with
      IsMeta n ->
          (try strip_outer_cast (List.assoc n metamap)
           with Not_found -> anomaly "type_of: this is not a well-typed term")
    | IsRel n -> lift n (body_of_type (snd (lookup_rel n env)))
    | IsVar id -> body_of_type (snd (lookup_var id env))

    | IsAbst _ -> error "No more Abst" (*type_of env (abst_value cstr)*)
    | IsConst c -> (body_of_type (type_of_constant env sigma c))
    | IsEvar _ -> type_of_existential env sigma cstr
    | IsMutInd ind -> (body_of_type (type_of_inductive env sigma ind))
    | IsMutConstruct cstr -> 
        let (typ,kind) = destCast (type_of_constructor env sigma cstr) in typ
    | IsMutCase (_,p,c,lf) ->
        let ind_data =
          try try_mutind_of env sigma (type_of env c)
          with Induc -> anomaly "type_of: Bad inductive" in
	let (aritysign,_) = get_arity env sigma ind_data in
	let (psign,_) = splay_prod env sigma (type_of env p) in
        let al =
	  if List.length psign > List.length aritysign
	  then ind_data.realargs@[c] else ind_data.realargs in
        whd_betadeltaiota env sigma (applist (p,al))
    | IsLambda (name,c1,c2) ->
        let var = make_typed c1 (sort_of env c1) in
          mkProd name c1 (type_of (push_rel (name,var) env) c2)
    | IsFix (vn,i,lar,lfi,vdef) -> lar.(i)
    | IsCoFix (i,lar,lfi,vdef) -> lar.(i)

    | IsAppL(f,args)-> strip_outer_cast (subst_type env sigma (type_of env f) args)
    | IsCast (c,t) -> t

    | IsSort _ | IsProd (_,_,_) | IsMutInd _ -> mkSort (sort_of env cstr)
    | _ -> error "type_of: Unexpected constr"

and sort_of env t = 
  match kind_of_term t with
    | IsCast (c,DOP0(Sort s)) -> s
    | IsSort (Prop c) -> type_0
    | IsSort (Type u) -> Type Univ.dummy_univ
    | IsProd (name,t,c2) ->
        let var = make_typed t (sort_of env t) in
        (match (sort_of (push_rel (name,var) env) c2) with
	  | Prop _ as s -> s
	  | Type u2 -> Type Univ.dummy_univ)
    | IsAppL(f,args) -> sort_of_atomic_type env sigma (type_of env f) args
    | IsLambda _ | IsFix _ | IsMutConstruct _ ->
        anomaly "sort_of: Not a type (1)"
    | _ -> outsort env sigma (type_of env t)

in type_of, sort_of

let get_type_of env sigma = fst (typeur sigma []) env
let get_sort_of env sigma = snd (typeur sigma []) env
let get_type_of_with_meta env sigma metamap = fst (typeur sigma metamap) env