package coq

  1. Overview
  2. Docs
On This Page
  1. Notations
Legend:
Library
Module
Module type
Parameter
Class
Class type
type context = (Names.Id.t * Tac2expr.type_scheme) list
val intern_open_type : Tac2expr.raw_typexpr -> Tac2expr.type_scheme
val is_value : Tac2expr.glb_tacexpr -> bool

Check that a term is a value. Only values are safe to marshall between processes.

val check_unit : ?loc:Loc.t -> Tac2expr.type_scheme -> unit
val check_subtype : Tac2expr.type_scheme -> Tac2expr.type_scheme -> bool

check_subtype t1 t2 returns true iff all values of instances of type t1 also have type t2.

Notations

Replaces all qualified identifiers by their corresponding kernel name. The set represents bound variables in the context.

Errors

val error_nargs_mismatch : ?loc:Loc.t -> Tac2expr.ltac_constructor -> int -> int -> 'a
val error_nparams_mismatch : ?loc:Loc.t -> int -> int -> 'a

Misc

val drop_ltac2_env : Genintern.Store.t -> Genintern.Store.t