package coq

  1. Overview
  2. Docs
Legend:
Page
Library
Module
Module type
Parameter
Class
Class type
Source

Module DetypingSource

Sourcetype _ delay =
  1. | Now : 'a delay
  2. | Later : [ `thunk ] delay
Sourceval print_universes : bool ref

Should we keep details of universes during detyping ?

Sourceval print_evar_arguments : bool ref

If true, prints full local context of evars

Sourceval print_factorize_match_patterns : unit -> bool

If true, contract branches with same r.h.s. and same matching variables in a disjunctive pattern

Sourceval print_allow_match_default_clause : unit -> bool

If this flag is true and the last non unique clause of a "match" is a variable-free disjunctive pattern, turn it into a catch-call case

Sourceval print_allow_match_default_opt_name : string list

detype isgoal avoid ctx c turns a closed c, into a glob_constr de Bruijn indexes are turned to bound names, avoiding names in avoid isgoal tells if naming must avoid global-level synonyms as intro does ctx gives the names of the free variables

Sourceval detype : 'a delay -> ?lax:bool -> bool -> Names.Id.Set.t -> Environ.env -> Evd.evar_map -> EConstr.constr -> 'a Glob_term.glob_constr_g
Sourceval detype_rel_context : 'a delay -> ?lax:bool -> EConstr.constr option -> Names.Id.Set.t -> (Termops.names_context * Environ.env) -> Evd.evar_map -> EConstr.rel_context -> 'a Glob_term.glob_decl_g list
Sourceval share_pattern_names : (Names.Id.Set.t -> Termops.names_context -> 'c -> Pattern.constr_pattern -> 'a) -> int -> (Names.Name.t * Glob_term.binding_kind * 'b option * 'a) list -> Names.Id.Set.t -> Termops.names_context -> 'c -> Pattern.constr_pattern -> Pattern.constr_pattern -> (Names.Name.t * Glob_term.binding_kind * 'b option * 'a) list * 'a * 'a
Sourceval lookup_name_as_displayed : Environ.env -> Evd.evar_map -> EConstr.constr -> Names.Id.t -> int option

look for the index of a named var or a nondep var as it is renamed

Sourceval lookup_index_as_renamed : Environ.env -> Evd.evar_map -> EConstr.constr -> int -> int option
Sourceval force_wildcard : unit -> bool
Sourceval synthetize_type : unit -> bool
Sourcemodule PrintingInductiveMake (Test : sig ... end) : sig ... end
OCaml

Innovation. Community. Security.