package coq
type lident = Names.Id.t Loc.located
type lname = Names.Name.t Loc.located
type lstring = string Loc.located
type goal_selector =
| SelectNth of int
| SelectList of (int * int) list
| SelectId of Names.Id.t
| SelectAll
type goal_reference =
| OpenSubgoals
| NthGoal of int
| GoalId of Names.Id.t
| GoalUid of goal_identifier
type printable =
| PrintTables
| PrintFullContext
| PrintSectionContext of Libnames.reference
| PrintInspect of int
| PrintGrammar of string
| PrintLoadPath of Names.DirPath.t option
| PrintModules
| PrintModule of Libnames.reference
| PrintModuleType of Libnames.reference
| PrintNamespace of Names.DirPath.t
| PrintMLLoadPath
| PrintMLModules
| PrintDebugGC
| PrintName of Libnames.reference Misctypes.or_by_notation
| PrintGraph
| PrintClasses
| PrintTypeClasses
| PrintInstances of Libnames.reference Misctypes.or_by_notation
| PrintCoercions
| PrintCoercionPaths of class_rawexpr * class_rawexpr
| PrintCanonicalConversions
| PrintUniverses of bool * string option
| PrintHint of Libnames.reference Misctypes.or_by_notation
| PrintHintGoal
| PrintHintDbName of string
| PrintHintDb
| PrintScopes
| PrintScope of string
| PrintVisibility of string option
| PrintAbout of Libnames.reference Misctypes.or_by_notation * goal_selector option
| PrintImplicit of Libnames.reference Misctypes.or_by_notation
| PrintAssumptions of bool * bool * Libnames.reference Misctypes.or_by_notation
| PrintStrategy of Libnames.reference Misctypes.or_by_notation option
type search_about_item =
| SearchSubPattern of Constrexpr.constr_pattern_expr
| SearchString of string * scope_name option
type searchable =
| SearchPattern of Constrexpr.constr_pattern_expr
| SearchRewrite of Constrexpr.constr_pattern_expr
| SearchHead of Constrexpr.constr_pattern_expr
| SearchAbout of (bool * search_about_item) list
type locatable =
| LocateAny of Libnames.reference Misctypes.or_by_notation
| LocateTerm of Libnames.reference Misctypes.or_by_notation
| LocateLibrary of Libnames.reference
| LocateModule of Libnames.reference
| LocateTactic of Libnames.reference
| LocateFile of string
type showable =
| ShowGoal of goal_reference
| ShowProof
| ShowScript
| ShowExistentials
| ShowUniverses
| ShowProofNames
| ShowIntros of bool
| ShowMatch of Libnames.reference
type comment =
| CommentConstr of Constrexpr.constr_expr
| CommentString of string
| CommentInt of int
type reference_or_constr =
| HintsReference of Libnames.reference
| HintsConstr of Constrexpr.constr_expr
type hint_info_expr = Constrexpr.constr_pattern_expr hint_info_gen
type hints_expr =
| HintsResolve of (hint_info_expr * bool * reference_or_constr) list
| HintsImmediate of reference_or_constr list
| HintsUnfold of Libnames.reference list
| HintsTransparency of Libnames.reference list * bool
| HintsMode of Libnames.reference * hint_mode list
| HintsConstructors of Libnames.reference list
| HintsExtern of int * Constrexpr.constr_expr option * Genarg.raw_generic_argument
type search_restriction =
| SearchInside of Libnames.reference list
| SearchOutside of Libnames.reference list
type inductive_flag = Decl_kinds.recursivity_kind
type onlyparsing_flag = Flags.compat_version option
type option_value = Goptions.option_value =
type sort_expr = Misctypes.glob_sort
type definition_expr =
| ProveBody of Constrexpr.local_binder_expr list * Constrexpr.constr_expr
| DefineBody of Constrexpr.local_binder_expr list * Genredexpr.raw_red_expr option * Constrexpr.constr_expr * Constrexpr.constr_expr option
type fixpoint_expr =
plident
* (Names.Id.t Loc.located option * Constrexpr.recursion_order_expr)
* Constrexpr.local_binder_expr list
* Constrexpr.constr_expr
* Constrexpr.constr_expr option
type cofixpoint_expr =
plident
* Constrexpr.local_binder_expr list
* Constrexpr.constr_expr
* Constrexpr.constr_expr option
type local_decl_expr =
| AssumExpr of lname * Constrexpr.constr_expr
| DefExpr of lname * Constrexpr.constr_expr * Constrexpr.constr_expr option
type decl_notation = lstring * Constrexpr.constr_expr * scope_name option
type simple_binder = lident list * Constrexpr.constr_expr
type class_binder = lident * Constrexpr.constr_expr list
type !'a with_coercion = coercion_flag * 'a
type !'a with_instance = instance_flag * 'a
type !'a with_notation = 'a * decl_notation list
type constructor_expr = (lident * Constrexpr.constr_expr) with_coercion
type constructor_list_or_record_decl_expr =
| Constructors of constructor_expr list
| RecordDecl of lident option * local_decl_expr with_instance with_priority with_notation list
type inductive_expr =
plident with_coercion
* Constrexpr.local_binder_expr list
* Constrexpr.constr_expr option
* inductive_kind
* constructor_list_or_record_decl_expr
type one_inductive_expr =
plident
* Constrexpr.local_binder_expr list
* Constrexpr.constr_expr option
* constructor_expr list
type proof_expr =
plident option * (Constrexpr.local_binder_expr list * Constrexpr.constr_expr)
type syntax_modifier =
| SetItemLevel of string list * Extend.production_level
| SetLevel of int
| SetAssoc of Extend.gram_assoc
| SetEntryType of string * Extend.simple_constr_prod_entry_key
| SetOnlyParsing
| SetOnlyPrinting
| SetCompatVersion of Flags.compat_version
| SetFormat of string * string Loc.located
type scheme =
| InductionScheme of bool * Libnames.reference Misctypes.or_by_notation * sort_expr
| CaseScheme of bool * Libnames.reference Misctypes.or_by_notation * sort_expr
| EqualityScheme of Libnames.reference Misctypes.or_by_notation
type section_subset_expr =
| SsEmpty
| SsSingl of lident
| SsCompl of section_subset_expr
| SsUnion of section_subset_expr * section_subset_expr
| SsSubstr of section_subset_expr * section_subset_expr
| SsFwdClose of section_subset_expr
type module_ast_inl = Constrexpr.module_ast * inline
type module_binder = bool option * lident list * module_ast_inl
type vernac_expr =
| VernacLoad of verbose_flag * string
| VernacTime of vernac_expr Loc.located
| VernacRedirect of string * vernac_expr Loc.located
| VernacTimeout of int * vernac_expr
| VernacFail of vernac_expr
| VernacSyntaxExtension of obsolete_locality * lstring * syntax_modifier list
| VernacOpenCloseScope of obsolete_locality * bool * scope_name
| VernacDelimiters of scope_name * string option
| VernacBindScope of scope_name * class_rawexpr list
| VernacInfix of obsolete_locality * lstring * syntax_modifier list * Constrexpr.constr_expr * scope_name option
| VernacNotation of obsolete_locality * Constrexpr.constr_expr * lstring * syntax_modifier list * scope_name option
| VernacNotationAddFormat of string * string * string
| VernacDefinition of Decl_kinds.locality option * Decl_kinds.definition_object_kind * plident * definition_expr
| VernacStartTheoremProof of Decl_kinds.theorem_kind * proof_expr list
| VernacEndProof of proof_end
| VernacExactProof of Constrexpr.constr_expr
| VernacAssumption of Decl_kinds.locality option * Decl_kinds.assumption_object_kind * inline * (plident list * Constrexpr.constr_expr) with_coercion list
| VernacInductive of cumulative_inductive_parsing_flag * Decl_kinds.private_flag * inductive_flag * (inductive_expr * decl_notation list) list
| VernacFixpoint of Decl_kinds.locality option * (fixpoint_expr * decl_notation list) list
| VernacCoFixpoint of Decl_kinds.locality option * (cofixpoint_expr * decl_notation list) list
| VernacScheme of (lident option * scheme) list
| VernacCombinedScheme of lident * lident list
| VernacUniverse of lident list
| VernacConstraint of (Misctypes.glob_level * Univ.constraint_type * Misctypes.glob_level) list
| VernacBeginSection of lident
| VernacEndSegment of lident
| VernacRequire of Libnames.reference option * export_flag option * Libnames.reference list
| VernacImport of export_flag * Libnames.reference list
| VernacCanonical of Libnames.reference Misctypes.or_by_notation
| VernacCoercion of obsolete_locality * Libnames.reference Misctypes.or_by_notation * class_rawexpr * class_rawexpr
| VernacIdentityCoercion of obsolete_locality * lident * class_rawexpr * class_rawexpr
| VernacNameSectionHypSet of lident * section_subset_expr
| VernacInstance of bool * Constrexpr.local_binder_expr list * Constrexpr.typeclass_constraint * (bool * Constrexpr.constr_expr) option * hint_info_expr
| VernacContext of Constrexpr.local_binder_expr list
| VernacDeclareInstances of (Libnames.reference * hint_info_expr) list
| VernacDeclareClass of Libnames.reference
| VernacDeclareModule of bool option * lident * module_binder list * module_ast_inl
| VernacDefineModule of bool option * lident * module_binder list * module_ast_inl module_signature * module_ast_inl list
| VernacDeclareModuleType of lident * module_binder list * module_ast_inl list * module_ast_inl list
| VernacInclude of module_ast_inl list
| VernacSolveExistential of int * Constrexpr.constr_expr
| VernacAddLoadPath of rec_flag * string * Names.DirPath.t option
| VernacRemoveLoadPath of string
| VernacAddMLPath of rec_flag * string
| VernacDeclareMLModule of string list
| VernacChdir of string option
| VernacWriteState of string
| VernacRestoreState of string
| VernacResetName of lident
| VernacResetInitial
| VernacBack of int
| VernacBackTo of int
| VernacCreateHintDb of string * bool
| VernacRemoveHints of string list * Libnames.reference list
| VernacHints of obsolete_locality * string list * hints_expr
| VernacSyntacticDefinition of Names.Id.t Loc.located * Names.Id.t list * Constrexpr.constr_expr * obsolete_locality * onlyparsing_flag
| VernacDeclareImplicits of Libnames.reference Misctypes.or_by_notation * (Constrexpr.explicitation * bool * bool) list list
| VernacArguments of Libnames.reference Misctypes.or_by_notation * vernac_argument_status list * (Names.Name.t * vernac_implicit_status) list list * int option * [ `Assert | `ClearImplicits | `ClearScopes | `DefaultImplicits | `ExtraScopes | `ReductionDontExposeCase | `ReductionNeverUnfold | `Rename ] list
| VernacArgumentsScope of Libnames.reference Misctypes.or_by_notation * scope_name option list
| VernacReserve of simple_binder list
| VernacGeneralizable of lident list option
| VernacSetOpacity of Conv_oracle.level * Libnames.reference Misctypes.or_by_notation list
| VernacSetStrategy of (Conv_oracle.level * Libnames.reference Misctypes.or_by_notation list) list
| VernacUnsetOption of Goptions.option_name
| VernacSetOption of Goptions.option_name * option_value
| VernacSetAppendOption of Goptions.option_name * string
| VernacAddOption of Goptions.option_name * option_ref_value list
| VernacRemoveOption of Goptions.option_name * option_ref_value list
| VernacMemOption of Goptions.option_name * option_ref_value list
| VernacPrintOption of Goptions.option_name
| VernacCheckMayEval of Genredexpr.raw_red_expr option * goal_selector option * Constrexpr.constr_expr
| VernacGlobalCheck of Constrexpr.constr_expr
| VernacDeclareReduction of string * Genredexpr.raw_red_expr
| VernacPrint of printable
| VernacSearch of searchable * goal_selector option * search_restriction
| VernacLocate of locatable
| VernacRegister of lident * register_kind
| VernacComments of comment list
| VernacStm of stm_vernac
| VernacGoal of Constrexpr.constr_expr
| VernacAbort of lident option
| VernacAbortAll
| VernacRestart
| VernacUndo of int
| VernacUndoTo of int
| VernacBacktrack of int * int * int
| VernacFocus of int option
| VernacUnfocus
| VernacUnfocused
| VernacBullet of bullet
| VernacSubproof of int option
| VernacEndSubproof
| VernacShow of showable
| VernacCheckGuard
| VernacProof of Genarg.raw_generic_argument option * section_subset_expr option
| VernacProofMode of string
| VernacToplevelControl of exn
| VernacExtend of extend_name * Genarg.raw_generic_argument list
| VernacProgram of vernac_expr
| VernacPolymorphic of bool * vernac_expr
| VernacLocal of bool * vernac_expr
and vernac_argument_status = {
name : Names.Name.t;
recarg_like : bool;
notation_scope : string Loc.located option;
implicit_status : vernac_implicit_status;
}
type vernac_type =
| VtStartProof of vernac_start
| VtSideff of vernac_sideff_type
| VtQed of vernac_qed_type
| VtProofStep of proof_step
| VtProofMode of string
| VtQuery of vernac_part_of_script * Feedback.route_id
| VtStm of vernac_control * vernac_part_of_script
| VtUnknown
and vernac_start = string * opacity_guarantee * Names.Id.t list
and vernac_sideff_type = Names.Id.t list
and proof_step = {
parallel : [ `No | `Yes of solving_tac * anon_abstracting_tac ];
proof_block_detection : proof_block_name option;
}
type vernac_classification = vernac_type * vernac_when
sectionYPositions = computeSectionYPositions($el), 10)"
x-init="setTimeout(() => sectionYPositions = computeSectionYPositions($el), 10)"
>