package coq

  1. Overview
  2. Docs
Legend:
Library
Module
Module type
Parameter
Class
Class type
type 'constr coeff_spec =
  1. | Computational of 'constr
  2. | Abstract
  3. | Morphism of 'constr
type cst_tac_spec =
  1. | CstTac of Ltac_plugin.Tacexpr.raw_tactic_expr
  2. | Closed of Libnames.qualid list
type 'constr ring_mod =
  1. | Ring_kind of 'constr coeff_spec
  2. | Const_tac of cst_tac_spec
  3. | Pre_tac of Ltac_plugin.Tacexpr.raw_tactic_expr
  4. | Post_tac of Ltac_plugin.Tacexpr.raw_tactic_expr
  5. | Setoid of Constrexpr.constr_expr * Constrexpr.constr_expr
  6. | Pow_spec of cst_tac_spec * Constrexpr.constr_expr
  7. | Sign_spec of Constrexpr.constr_expr
  8. | Div_spec of Constrexpr.constr_expr
type 'constr field_mod =
  1. | Ring_mod of 'constr ring_mod
  2. | Inject of Constrexpr.constr_expr
type ring_info = {
  1. ring_name : Names.Id.t;
  2. ring_carrier : Constr.types;
  3. ring_req : Constr.constr;
  4. ring_setoid : Constr.constr;
  5. ring_ext : Constr.constr;
  6. ring_morph : Constr.constr;
  7. ring_th : Constr.constr;
  8. ring_cst_tac : Ltac_plugin.Tacexpr.glob_tactic_expr;
  9. ring_pow_tac : Ltac_plugin.Tacexpr.glob_tactic_expr;
  10. ring_lemma1 : Constr.constr;
  11. ring_lemma2 : Constr.constr;
  12. ring_pre_tac : Ltac_plugin.Tacexpr.glob_tactic_expr;
  13. ring_post_tac : Ltac_plugin.Tacexpr.glob_tactic_expr;
}
type field_info = {
  1. field_name : Names.Id.t;
  2. field_carrier : Constr.types;
  3. field_req : Constr.constr;
  4. field_cst_tac : Ltac_plugin.Tacexpr.glob_tactic_expr;
  5. field_pow_tac : Ltac_plugin.Tacexpr.glob_tactic_expr;
  6. field_ok : Constr.constr;
  7. field_simpl_eq_ok : Constr.constr;
  8. field_simpl_ok : Constr.constr;
  9. field_simpl_eq_in_ok : Constr.constr;
  10. field_cond : Constr.constr;
  11. field_pre_tac : Ltac_plugin.Tacexpr.glob_tactic_expr;
  12. field_post_tac : Ltac_plugin.Tacexpr.glob_tactic_expr;
}