diff --git a/master/api/coq-core/DeclareUniv/index.html b/master/api/coq-core/DeclareUniv/index.html index ebf7ecb85f..550bc77b20 100644 --- a/master/api/coq-core/DeclareUniv/index.html +++ b/master/api/coq-core/DeclareUniv/index.html @@ -1,2 +1,2 @@ -DeclareUniv (coq-core.DeclareUniv)

Module DeclareUniv

exception AlreadyDeclared of string option * Names.Id.t

Also used by Declare for constants, DeclareInd for inductives, etc. Containts object_kind , id.

val declare_univ_binders : Names.GlobRef.t -> UState.named_universes_entry -> unit

Internally used to declare names of universes from monomorphic constants/inductives. Noop on polymorphic references.

val do_universe : poly:bool -> Names.lident list -> unit

Command Universes.

val do_constraint : poly:bool -> Constrexpr.univ_constraint_expr list -> unit

Command Constraint.

val add_constraint_source : Names.GlobRef.t -> Univ.ContextSet.t -> unit
val constraint_sources : unit -> (Names.GlobRef.t * Univ.Constraints.t) list

Returns constraints associated to globrefs, newest first.

\ No newline at end of file +DeclareUniv (coq-core.DeclareUniv)

Module DeclareUniv

exception AlreadyDeclared of string option * Names.Id.t

Also used by Declare for constants, DeclareInd for inductives, etc. Containts object_kind , id.

val declare_univ_binders : Names.GlobRef.t -> UState.named_universes_entry -> unit

Internally used to declare names of universes from monomorphic constants/inductives. Noop on polymorphic references.

val name_mono_section_univs : Univ.Level.Set.t -> unit

Internally used to name universes associated with no particular constant in a section.

val do_universe : poly:bool -> Names.lident list -> unit

Command Universes.

val do_constraint : poly:bool -> Constrexpr.univ_constraint_expr list -> unit

Command Constraint.

val add_constraint_source : Names.GlobRef.t -> Univ.ContextSet.t -> unit
val constraint_sources : unit -> (Names.GlobRef.t * Univ.Constraints.t) list

Returns constraints associated to globrefs, newest first.

\ No newline at end of file diff --git a/master/api/coq-core/Lib/Interp/index.html b/master/api/coq-core/Lib/Interp/index.html index 2b7e681b2e..2b70310ddb 100644 --- a/master/api/coq-core/Lib/Interp/index.html +++ b/master/api/coq-core/Lib/Interp/index.html @@ -1,2 +1,2 @@ -Interp (coq-core.Lib.Interp)

Module Lib.Interp

type summary = Summary.Interp.frozen
type classified_objects = {
substobjs : Libobject.t list;
keepobjs : Libobject.t list;
anticipateobjs : Libobject.t list;
}
val classify_segment : Libobject.t list -> classified_objects
val find_opening_node : ?loc:Loc.t -> Names.Id.t -> summary node

Returns the opening node of a given name

val add_entry : summary node -> unit
val add_leaf_entry : Libobject.t -> unit
val open_section : Names.Id.t -> unit

Sections

val close_section : unit -> discharged_item list

close_section needs to redo Export, so the complete implementation needs to involve Declaremods.

Modules and module types
val end_module : unit -> Nametab.object_prefix * summary * classified_objects
val end_modtype : unit -> Nametab.object_prefix * summary * classified_objects
type frozen
val freeze : unit -> frozen
val unfreeze : frozen -> unit
val init : unit -> unit
val drop_objects : frozen -> frozen

Keep only the libobject structure, not the objects themselves

val declare_info : Library_info.t -> unit
\ No newline at end of file +Interp (coq-core.Lib.Interp)

Module Lib.Interp

type summary = Summary.Interp.frozen
val find_opening_node : ?loc:Loc.t -> Names.Id.t -> summary node

Returns the opening node of a given name

val add_entry : summary node -> unit
val add_leaf_entry : Libobject.t -> unit
val open_section : Names.Id.t -> unit

Sections

val close_section : unit -> discharged_item list

close_section needs to redo Export, so the complete implementation needs to involve Declaremods.

Modules and module types
val end_module : unit -> Nametab.object_prefix * summary * classified_objects
val end_modtype : unit -> Nametab.object_prefix * summary * classified_objects
type frozen
val freeze : unit -> frozen
val unfreeze : frozen -> unit
val init : unit -> unit
val drop_objects : frozen -> frozen

Keep only the libobject structure, not the objects themselves

val declare_info : Library_info.t -> unit
\ No newline at end of file diff --git a/master/api/coq-core/Lib/Synterp/index.html b/master/api/coq-core/Lib/Synterp/index.html index 6bb6a02f68..ee3c580b43 100644 --- a/master/api/coq-core/Lib/Synterp/index.html +++ b/master/api/coq-core/Lib/Synterp/index.html @@ -1,2 +1,2 @@ -Synterp (coq-core.Lib.Synterp)

Module Lib.Synterp

type summary = Summary.Synterp.frozen
type classified_objects = {
substobjs : Libobject.t list;
keepobjs : Libobject.t list;
anticipateobjs : Libobject.t list;
}
val classify_segment : Libobject.t list -> classified_objects
val find_opening_node : ?loc:Loc.t -> Names.Id.t -> summary node

Returns the opening node of a given name

val add_entry : summary node -> unit
val add_leaf_entry : Libobject.t -> unit
val open_section : Names.Id.t -> unit

Sections

val close_section : unit -> discharged_item list

close_section needs to redo Export, so the complete implementation needs to involve Declaremods.

Modules and module types
val end_module : unit -> Nametab.object_prefix * summary * classified_objects
val end_modtype : unit -> Nametab.object_prefix * summary * classified_objects
type frozen
val freeze : unit -> frozen
val unfreeze : frozen -> unit
val init : unit -> unit
val drop_objects : frozen -> frozen

Keep only the libobject structure, not the objects themselves

val declare_info : Library_info.t -> unit
\ No newline at end of file +Synterp (coq-core.Lib.Synterp)

Module Lib.Synterp

type summary = Summary.Synterp.frozen
val find_opening_node : ?loc:Loc.t -> Names.Id.t -> summary node

Returns the opening node of a given name

val add_entry : summary node -> unit
val add_leaf_entry : Libobject.t -> unit
val open_section : Names.Id.t -> unit

Sections

val close_section : unit -> discharged_item list

close_section needs to redo Export, so the complete implementation needs to involve Declaremods.

Modules and module types
val end_module : unit -> Nametab.object_prefix * summary * classified_objects
val end_modtype : unit -> Nametab.object_prefix * summary * classified_objects
type frozen
val freeze : unit -> frozen
val unfreeze : frozen -> unit
val init : unit -> unit
val drop_objects : frozen -> frozen

Keep only the libobject structure, not the objects themselves

val declare_info : Library_info.t -> unit
\ No newline at end of file diff --git a/master/api/coq-core/Lib/index.html b/master/api/coq-core/Lib/index.html index 5c06f8ec68..be5ac3d404 100644 --- a/master/api/coq-core/Lib/index.html +++ b/master/api/coq-core/Lib/index.html @@ -1,2 +1,2 @@ -Lib (coq-core.Lib)

Module Lib

Lib: record of operations, backtrack, low-level sections

This module provides a general mechanism to keep a trace of all operations and to backtrack (undo) those operations. It provides also the section mechanism (at a low level; discharge is not known at this step).

type is_type = bool
type export_flag =
| Export
| Import
type export = (export_flag * Libobject.open_filter) option
val make_foname : Names.Id.t -> Libobject.object_name
type 'summary node =
| CompilingLibrary of Nametab.object_prefix
| OpenedModule of is_type * export * Nametab.object_prefix * 'summary
| OpenedSection of Nametab.object_prefix * 'summary
val node_prefix : 'summary node -> Nametab.object_prefix

Extract the object_prefix component. Note that it is the prefix of the objects *inside* this node, eg in Module M. we have OpenedModule with prefix containing M.

type 'summary library_segment = ('summary node * Libobject.t list) list
...

Adding operations (which call the cache method, and getting the current list of operations (most recent ones coming first).

val add_leaf : Libobject.obj -> unit
val add_discharged_leaf : Libobject.discharged_obj -> unit
...

The function contents gives access to the current entire segment

val contents : unit -> Summary.Interp.frozen library_segment
Functions relative to current path
val prefix : unit -> Nametab.object_prefix

User-side names

cwd() is (prefix()).obj_dir current_mp() is (prefix()).obj_mp

Inside a library A.B module M section S, we have

  • library_dp = A.B
  • cwd = A.B.M.S
  • cwd_except_section = A.B.M
  • current_dirpath true = M.S
  • current_dirpath false = S
  • current_mp = MPdot(MPfile A.B, M)

make_path (resp make_path_except_section) uses cwd (resp cwd_except_section) make_kn uses current_mp

val cwd : unit -> Names.DirPath.t
val cwd_except_section : unit -> Names.DirPath.t
val current_dirpath : bool -> Names.DirPath.t
val make_path : Names.Id.t -> Libnames.full_path
val make_path_except_section : Names.Id.t -> Libnames.full_path
val current_mp : unit -> Names.ModPath.t

Kernel-side names

val make_kn : Names.Id.t -> Names.KerName.t
val sections_are_opened : unit -> bool

Are we inside an opened section

val sections_depth : unit -> int
val is_module_or_modtype : unit -> bool

Are we inside an opened module type

val is_modtype : unit -> bool
val is_modtype_strict : unit -> bool
val is_module : unit -> bool
type discharged_item =
| DischargedExport of Libobject.ExportObj.t
| DischargedLeaf of Libobject.discharged_obj
module type StagedLibS = sig ... end

The StagedLibS abstraction describes operations and traversal for Lib at a given stage.

We provide two instances of StagedLibS, corresponding to the Synterp and Interp stages.

Compilation units
val start_compilation : Names.DirPath.t -> Names.ModPath.t -> unit

Finalize the compilation of a library and return respectively the library prefix, the regular objects, and the syntax-related objects.

val library_dp : unit -> Names.DirPath.t

The function library_dp returns the DirPath.t of the current compiling library (or default_library)

val split_modpath : Names.ModPath.t -> Names.DirPath.t * Names.Id.t list

Extract the library part of a name even if in a section

val library_part : Names.GlobRef.t -> Names.DirPath.t
val section_segment_of_constant : Names.Constant.t -> Cooking.cooking_info

Section management for discharge

val section_segment_of_inductive : Names.MutInd.t -> Cooking.cooking_info
val section_segment_of_reference : Names.GlobRef.t -> Cooking.cooking_info
val section_instance : Names.GlobRef.t -> Constr.t array
val is_in_section : Names.GlobRef.t -> bool
Discharge: decrease the section level if in the current section

discharge_proj_repr p discharges projection p if the associated record was defined in the current section. If that is not the case, it returns p unchanged.

Compatibility layer

val init : unit -> unit

This also does init_summaries

\ No newline at end of file +Lib (coq-core.Lib)

Module Lib

Lib: record of operations, backtrack, low-level sections

This module provides a general mechanism to keep a trace of all operations and to backtrack (undo) those operations. It provides also the section mechanism (at a low level; discharge is not known at this step).

type is_type = bool
type export_flag =
| Export
| Import
type export = (export_flag * Libobject.open_filter) option
val make_foname : Names.Id.t -> Libobject.object_name
type 'summary node =
| CompilingLibrary of Nametab.object_prefix
| OpenedModule of is_type * export * Nametab.object_prefix * 'summary
| OpenedSection of Nametab.object_prefix * 'summary
val node_prefix : 'summary node -> Nametab.object_prefix

Extract the object_prefix component. Note that it is the prefix of the objects *inside* this node, eg in Module M. we have OpenedModule with prefix containing M.

type 'summary library_segment = ('summary node * Libobject.t list) list
...

Adding operations (which call the cache method, and getting the current list of operations (most recent ones coming first).

val add_leaf : Libobject.obj -> unit
val add_discharged_leaf : Libobject.discharged_obj -> unit
...

The function contents gives access to the current entire segment

val contents : unit -> Summary.Interp.frozen library_segment
Functions relative to current path
val prefix : unit -> Nametab.object_prefix

User-side names

cwd() is (prefix()).obj_dir current_mp() is (prefix()).obj_mp

Inside a library A.B module M section S, we have

  • library_dp = A.B
  • cwd = A.B.M.S
  • cwd_except_section = A.B.M
  • current_dirpath true = M.S
  • current_dirpath false = S
  • current_mp = MPdot(MPfile A.B, M)

make_path (resp make_path_except_section) uses cwd (resp cwd_except_section) make_kn uses current_mp

val cwd : unit -> Names.DirPath.t
val cwd_except_section : unit -> Names.DirPath.t
val current_dirpath : bool -> Names.DirPath.t
val make_path : Names.Id.t -> Libnames.full_path
val make_path_except_section : Names.Id.t -> Libnames.full_path
val current_mp : unit -> Names.ModPath.t

Kernel-side names

val make_kn : Names.Id.t -> Names.KerName.t
val sections_are_opened : unit -> bool

Are we inside an opened section

val sections_depth : unit -> int
val is_module_or_modtype : unit -> bool

Are we inside an opened module type

val is_modtype : unit -> bool
val is_modtype_strict : unit -> bool
val is_module : unit -> bool
type discharged_item =
| DischargedExport of Libobject.ExportObj.t
| DischargedLeaf of Libobject.discharged_obj
type classified_objects = {
substobjs : Libobject.t list;
keepobjs : Libobject.t list;
escapeobjs : Libobject.t list;
anticipateobjs : Libobject.t list;
}
module type StagedLibS = sig ... end

The StagedLibS abstraction describes operations and traversal for Lib at a given stage.

We provide two instances of StagedLibS, corresponding to the Synterp and Interp stages.

Compilation units
val start_compilation : Names.DirPath.t -> Names.ModPath.t -> unit
type compilation_result = {
info : Library_info.t;
synterp_objects : classified_objects;
interp_objects : classified_objects;
}
val end_compilation : Names.DirPath.t -> compilation_result

Finalize the compilation of a library.

val library_dp : unit -> Names.DirPath.t

The function library_dp returns the DirPath.t of the current compiling library (or default_library)

val split_modpath : Names.ModPath.t -> Names.DirPath.t * Names.Id.t list

Extract the library part of a name even if in a section

val library_part : Names.GlobRef.t -> Names.DirPath.t
val section_segment_of_constant : Names.Constant.t -> Cooking.cooking_info

Section management for discharge

val section_segment_of_inductive : Names.MutInd.t -> Cooking.cooking_info
val section_segment_of_reference : Names.GlobRef.t -> Cooking.cooking_info
val section_instance : Names.GlobRef.t -> Constr.t array
val is_in_section : Names.GlobRef.t -> bool
Discharge: decrease the section level if in the current section

discharge_proj_repr p discharges projection p if the associated record was defined in the current section. If that is not the case, it returns p unchanged.

Compatibility layer

val init : unit -> unit

This also does init_summaries

\ No newline at end of file diff --git a/master/api/coq-core/Lib/module-type-StagedLibS/index.html b/master/api/coq-core/Lib/module-type-StagedLibS/index.html index 105133444a..35a351f28c 100644 --- a/master/api/coq-core/Lib/module-type-StagedLibS/index.html +++ b/master/api/coq-core/Lib/module-type-StagedLibS/index.html @@ -1,2 +1,2 @@ -StagedLibS (coq-core.Lib.StagedLibS)

Module type Lib.StagedLibS

The StagedLibS abstraction describes operations and traversal for Lib at a given stage.

type summary
type classified_objects = {
substobjs : Libobject.t list;
keepobjs : Libobject.t list;
anticipateobjs : Libobject.t list;
}
val classify_segment : Libobject.t list -> classified_objects
val find_opening_node : ?loc:Loc.t -> Names.Id.t -> summary node

Returns the opening node of a given name

val add_entry : summary node -> unit
val add_leaf_entry : Libobject.t -> unit
val open_section : Names.Id.t -> unit

Sections

val close_section : unit -> discharged_item list

close_section needs to redo Export, so the complete implementation needs to involve Declaremods.

Modules and module types
val end_module : unit -> Nametab.object_prefix * summary * classified_objects
val end_modtype : unit -> Nametab.object_prefix * summary * classified_objects
type frozen
val freeze : unit -> frozen
val unfreeze : frozen -> unit
val init : unit -> unit
val drop_objects : frozen -> frozen

Keep only the libobject structure, not the objects themselves

val declare_info : Library_info.t -> unit
\ No newline at end of file +StagedLibS (coq-core.Lib.StagedLibS)

Module type Lib.StagedLibS

The StagedLibS abstraction describes operations and traversal for Lib at a given stage.

type summary
val find_opening_node : ?loc:Loc.t -> Names.Id.t -> summary node

Returns the opening node of a given name

val add_entry : summary node -> unit
val add_leaf_entry : Libobject.t -> unit
val open_section : Names.Id.t -> unit

Sections

val close_section : unit -> discharged_item list

close_section needs to redo Export, so the complete implementation needs to involve Declaremods.

Modules and module types
val end_module : unit -> Nametab.object_prefix * summary * classified_objects
val end_modtype : unit -> Nametab.object_prefix * summary * classified_objects
type frozen
val freeze : unit -> frozen
val unfreeze : frozen -> unit
val init : unit -> unit
val drop_objects : frozen -> frozen

Keep only the libobject structure, not the objects themselves

val declare_info : Library_info.t -> unit
\ No newline at end of file diff --git a/master/api/coq-core/Libobject/index.html b/master/api/coq-core/Libobject/index.html index efebb19ef4..046ef969b3 100644 --- a/master/api/coq-core/Libobject/index.html +++ b/master/api/coq-core/Libobject/index.html @@ -1,7 +1,7 @@ -Libobject (coq-core.Libobject)

Module Libobject

Libobject declares persistent objects, given with methods:

* a caching function specifying how to add the object in the current scope; called when the object is added and after the end of the containing sections. If the object wishes to register its visibility in the Nametab, it should do so for all possible suffixes.

* a loading function, specifying what to do when the module containing the object is loaded; called at Require and after the end of the containing modules. If the object wishes to register its visibility in the Nametab, it should do so for all suffixes no shorter than the "int" argument

* an opening function, specifying what to do when the module containing the object is opened; called when the containing modules are Imported. Objects which should only have an effect when the nearest containing module is imported (and not when the modules containing the nearest module are imported) must check that the "int" argument is 1. If the object wishes to register its visibility in the Nametab, it should do so for the suffix of the length the "int" argument

* a classification function, specifying what to do with the object, when the current module (containing the object) is ended; The possibilities are: Dispose - the object is dropped at the end of the module. Substitute - the object is kept at the end of the module. When the module is cloned (Include, module aliases) or when it's a module type which is getting instantiated (eg if module type T is used for a functor argument X : T or Declare Module X : T), the substitution function is called on the object to update the module name. Keep - the object is kept at the end of the module. When the module is cloned the object is not cloned with it. This means that Keep objects in a module type or functor are dropped. Anticipate - this is for objects that have to be explicitly managed by the end_module function (currently only Require).

* a substitution function, performing the substitution; this function should be declared for substitutive objects only (see above). NB: the substitution might be delayed instead of happening at module creation, so this function should _not_ depend on the current environment

* a discharge function, that is called at section closing time to collect the data necessary to rebuild the discharged form of the non volatile objects. If it returns None the object is dropped. It is called in the state inside the section at its end, before it is reset. Notably the global environment contains the section data and the non-discharged globals.

* a rebuild function, that is applied after section closing to rebuild the non volatile content of a section from the data collected by the discharge function It is called in the state after the end of the section with any previous objects already present. Notably the global environment contains the discharged globals.

Any type defined as a persistent object must be pure (e.g. no references) and marshallable by the OCaml Marshal module (e.g. no closures).

type substitutivity =
| Dispose
| Substitute
| Keep
| Anticipate

Both names are passed to objects: a "semantic" kernel_name, which can be substituted and a "syntactic" full_path which can be printed

type object_name = Libnames.full_path * Names.KerName.t
type open_filter
type ('a, 'b, 'discharged) object_declaration = {
object_name : string;
object_stage : Summary.Stage.t;
cache_function : 'b -> unit;
load_function : int -> 'b -> unit;
open_function : open_filter -> int -> 'b -> unit;
classify_function : 'a -> substitutivity;
subst_function : (Mod_subst.substitution * 'a) -> 'a;
discharge_function : 'a -> 'discharged option;
rebuild_function : 'discharged -> 'a;
}
val unfiltered : open_filter
val make_filter : finite:bool -> string CAst.t list -> open_filter

Anomaly when the list is empty.

type category
val create_category : string -> category

Anomaly if called more than once for a given string.

val in_filter : cat:category option -> open_filter -> bool

On cat:None, returns whether the filter allows opening uncategorized objects.

On cat:(Some category), returns whether the filter allows opening objects in the given category.

val simple_open : ?cat:category -> ('i -> 'a -> unit) -> open_filter -> 'i -> 'a -> unit

Combinator for making objects with simple category-based open behaviour. When cat:None, can be opened by Unfiltered, but also by Filtered with a negative set.

val filter_eq : open_filter -> open_filter -> bool
val filter_and : open_filter -> open_filter -> open_filter option

Returns None when the intersection is empty.

val filter_or : open_filter -> open_filter -> open_filter

The default object is a "Keep" object with empty methods. Object creators are advised to use the construction {(default_object "MY_OBJECT") with +Libobject (coq-core.Libobject)

Module Libobject

Libobject declares persistent objects, given with methods:

* a caching function specifying how to add the object in the current scope; called when the object is added and after the end of the containing sections. If the object wishes to register its visibility in the Nametab, it should do so for all possible suffixes.

* a loading function, specifying what to do when the module containing the object is loaded; called at Require and after the end of the containing modules. If the object wishes to register its visibility in the Nametab, it should do so for all suffixes no shorter than the "int" argument

* an opening function, specifying what to do when the module containing the object is opened; called when the containing modules are Imported. Objects which should only have an effect when the nearest containing module is imported (and not when the modules containing the nearest module are imported) must check that the "int" argument is 1. If the object wishes to register its visibility in the Nametab, it should do so for the suffix of the length the "int" argument

* a classification function, specifying what to do with the object, when the current module (containing the object) is ended; The possibilities are: Dispose - the object is dropped at the end of the module. Substitute - the object is kept at the end of the module. When the module is cloned (Include, module aliases) or when it's a module type which is getting instantiated (eg if module type T is used for a functor argument X : T or Declare Module X : T), the substitution function is called on the object to update the module name. Keep - the object is kept at the end of the module. When the module is cloned the object is not cloned with it. This means that Keep objects in a module type or functor are dropped. Escape - like Keep, but also escapes module types, functors and opaque modules. Monomorphic universes and universe constraints behave like this. Anticipate - this is for objects that have to be explicitly managed by the end_module function (currently only Require).

* a substitution function, performing the substitution; this function should be declared for substitutive objects only (see above). NB: the substitution might be delayed instead of happening at module creation, so this function should _not_ depend on the current environment

* a discharge function, that is called at section closing time to collect the data necessary to rebuild the discharged form of the non volatile objects. If it returns None the object is dropped. It is called in the state inside the section at its end, before it is reset. Notably the global environment contains the section data and the non-discharged globals.

* a rebuild function, that is applied after section closing to rebuild the non volatile content of a section from the data collected by the discharge function It is called in the state after the end of the section with any previous objects already present. Notably the global environment contains the discharged globals.

Any type defined as a persistent object must be pure (e.g. no references) and marshallable by the OCaml Marshal module (e.g. no closures).

type substitutivity =
| Dispose
| Substitute
| Keep
| Escape
| Anticipate

Both names are passed to objects: a "semantic" kernel_name, which can be substituted and a "syntactic" full_path which can be printed

type object_name = Libnames.full_path * Names.KerName.t
type open_filter
type ('a, 'b, 'discharged) object_declaration = {
object_name : string;
object_stage : Summary.Stage.t;
cache_function : 'b -> unit;
load_function : int -> 'b -> unit;
open_function : open_filter -> int -> 'b -> unit;
classify_function : 'a -> substitutivity;
subst_function : (Mod_subst.substitution * 'a) -> 'a;
discharge_function : 'a -> 'discharged option;
rebuild_function : 'discharged -> 'a;
}
val unfiltered : open_filter
val make_filter : finite:bool -> string CAst.t list -> open_filter

Anomaly when the list is empty.

type category
val create_category : string -> category

Anomaly if called more than once for a given string.

val in_filter : cat:category option -> open_filter -> bool

On cat:None, returns whether the filter allows opening uncategorized objects.

On cat:(Some category), returns whether the filter allows opening objects in the given category.

val simple_open : ?cat:category -> ('i -> 'a -> unit) -> open_filter -> 'i -> 'a -> unit

Combinator for making objects with simple category-based open behaviour. When cat:None, can be opened by Unfiltered, but also by Filtered with a negative set.

val filter_eq : open_filter -> open_filter -> bool
val filter_and : open_filter -> open_filter -> open_filter option

Returns None when the intersection is empty.

val filter_or : open_filter -> open_filter -> open_filter

The default object has empty methods. Object creators are advised to use the construction {(default_object "MY_OBJECT") with cache_function = ... - } and specify only these functions which are not empty/meaningless

val default_object : ?stage:Summary.Stage.t -> string -> ('a'b'a) object_declaration
val ident_subst_function : (Mod_subst.substitution * 'a) -> 'a

the identity substitution function

...

Given an object declaration, the function declare_object_full will hand back two functions, the "injection" and "projection" functions for dynamically typed library-objects.

module Dyn : Dyn.S
type obj = Dyn.t
module ExportObj : sig ... end
type algebraic_objects =
| Objs of t list
| Ref of Names.ModPath.t * Mod_subst.substitution
and t =
| ModuleObject of Names.Id.t * substitutive_objects
| ModuleTypeObject of Names.Id.t * substitutive_objects
| IncludeObject of algebraic_objects
| KeepObject of Names.Id.t * t list
| ExportObject of ExportObj.t
| AtomicObject of obj
and substitutive_objects = Names.MBId.t list * algebraic_objects

Object declaration and names: if you need the current prefix (typically to interact with the nametab), you need to have it passed to you.

val declare_object : ('a'a_) object_declaration -> 'a -> obj
val declare_object_full : ('a'a_) object_declaration -> 'a Dyn.tag
val declare_named_object_full : ('aobject_name * 'a_) object_declaration -> (Names.Id.t * 'a) Dyn.tag
val declare_named_object : ('aobject_name * 'a_) object_declaration -> Names.Id.t -> 'a -> obj
val declare_named_object_gen : ('aNametab.object_prefix * 'a_) object_declaration -> 'a -> obj
val cache_object : (Nametab.object_prefix * obj) -> unit
val load_object : int -> (Nametab.object_prefix * obj) -> unit
val open_object : open_filter -> int -> (Nametab.object_prefix * obj) -> unit
val subst_object : (Mod_subst.substitution * obj) -> obj
val classify_object : obj -> substitutivity
val object_stage : obj -> Summary.Stage.t
type discharged_obj
val discharge_object : obj -> discharged_obj option
val rebuild_object : discharged_obj -> obj
type locality =
| Local
| Export
| SuperGlobal
val object_with_locality : ?stage:Summary.Stage.t -> ?cat:category -> string -> cache:('a -> unit) -> + } and specify only these functions which are not empty/meaningless

The classify_function must be specified.

val default_object : ?stage:Summary.Stage.t -> string -> ('a'b'a) object_declaration
val ident_subst_function : (Mod_subst.substitution * 'a) -> 'a

the identity substitution function

...

Given an object declaration, the function declare_object_full will hand back two functions, the "injection" and "projection" functions for dynamically typed library-objects.

module Dyn : Dyn.S
type obj = Dyn.t
module ExportObj : sig ... end
type algebraic_objects =
| Objs of t list
| Ref of Names.ModPath.t * Mod_subst.substitution
and t =
| ModuleObject of Names.Id.t * substitutive_objects
| ModuleTypeObject of Names.Id.t * substitutive_objects
| IncludeObject of algebraic_objects
| KeepObject of Names.Id.t * t list
| EscapeObject of Names.Id.t * t list
| ExportObject of ExportObj.t
| AtomicObject of obj
and substitutive_objects = Names.MBId.t list * algebraic_objects

Object declaration and names: if you need the current prefix (typically to interact with the nametab), you need to have it passed to you.

  • declare_named_object_gen passes the raw prefix which you can manipulate as you wish.
  • declare_named_object_full and declare_named_object provide the convenience of packaging it with the provided Id.t into a object_name.
  • declare_object and declare_object_full ignore the prefix for you.
val declare_object : ('a'a_) object_declaration -> 'a -> obj
val declare_object_full : ('a'a_) object_declaration -> 'a Dyn.tag
val declare_named_object_full : ('aobject_name * 'a_) object_declaration -> (Names.Id.t * 'a) Dyn.tag
val declare_named_object : ('aobject_name * 'a_) object_declaration -> Names.Id.t -> 'a -> obj
val declare_named_object_gen : ('aNametab.object_prefix * 'a_) object_declaration -> 'a -> obj
val cache_object : (Nametab.object_prefix * obj) -> unit
val load_object : int -> (Nametab.object_prefix * obj) -> unit
val open_object : open_filter -> int -> (Nametab.object_prefix * obj) -> unit
val subst_object : (Mod_subst.substitution * obj) -> obj
val classify_object : obj -> substitutivity
val object_stage : obj -> Summary.Stage.t
type discharged_obj
val discharge_object : obj -> discharged_obj option
val rebuild_object : discharged_obj -> obj
type locality =
| Local
| Export
| SuperGlobal
val object_with_locality : ?stage:Summary.Stage.t -> ?cat:category -> string -> cache:('a -> unit) -> subst:((Mod_subst.substitution * 'a) -> 'a) option -> discharge:('a -> 'a) -> (locality * 'alocality * 'alocality * 'a) object_declaration

Object with semi-static scoping: the scoping depends on the given locality not the rest of the object.

It is up to the caller of add_leaf to produce sensible errors if a value which cannot be discharged is given with non Local locality.

If subst is None non Local values are Keep, otherwise Substitute.

Export values are only imported with shallow imports (depth = 1).

cat only matters when importing, ie only for Export values.

Higher-level API for objects with fixed scope.

  • Local means that the object cannot be imported from outside.
  • Global means that it can be imported (by importing the module that contains the object).
  • Superglobal means that the object survives to closing a module, and is imported when the file which contains it is Required (even without Import).
  • With the nodischarge variants, the object does not survive section closing. With the normal variants, it does.

We recommend to avoid declaring superglobal objects and using the nodischarge variants.

val local_object : ?stage:Summary.Stage.t -> string -> cache:('a -> unit) -> discharge:('a -> 'a option) -> ('a'a'a) object_declaration
val local_object_nodischarge : ?stage:Summary.Stage.t -> string -> cache:('a -> unit) -> ('a'a'a) object_declaration
val global_object : ?cat:category -> ?stage:Summary.Stage.t -> string -> cache:('a -> unit) -> diff --git a/master/refman/.doctrees/addendum/generalized-rewriting.doctree b/master/refman/.doctrees/addendum/generalized-rewriting.doctree index 1df617c901..12da6e8521 100644 Binary files a/master/refman/.doctrees/addendum/generalized-rewriting.doctree and b/master/refman/.doctrees/addendum/generalized-rewriting.doctree differ diff --git a/master/refman/.doctrees/addendum/universe-polymorphism.doctree b/master/refman/.doctrees/addendum/universe-polymorphism.doctree index 4d62c795ca..2c9ecdeda5 100644 Binary files a/master/refman/.doctrees/addendum/universe-polymorphism.doctree and b/master/refman/.doctrees/addendum/universe-polymorphism.doctree differ diff --git a/master/refman/.doctrees/environment.pickle b/master/refman/.doctrees/environment.pickle index 6a7454c694..d146f8fc2e 100644 Binary files a/master/refman/.doctrees/environment.pickle and b/master/refman/.doctrees/environment.pickle differ diff --git a/master/refman/.doctrees/language/coq-library.doctree b/master/refman/.doctrees/language/coq-library.doctree index 9fe1292b42..06c6fd1263 100644 Binary files a/master/refman/.doctrees/language/coq-library.doctree and b/master/refman/.doctrees/language/coq-library.doctree differ diff --git a/master/refman/.doctrees/language/core/conversion.doctree b/master/refman/.doctrees/language/core/conversion.doctree index 629fdf126a..9a41addcef 100644 Binary files a/master/refman/.doctrees/language/core/conversion.doctree and b/master/refman/.doctrees/language/core/conversion.doctree differ diff --git a/master/refman/.doctrees/language/core/modules.doctree b/master/refman/.doctrees/language/core/modules.doctree index f59d69a4c0..9538a42304 100644 Binary files a/master/refman/.doctrees/language/core/modules.doctree and b/master/refman/.doctrees/language/core/modules.doctree differ diff --git a/master/refman/.doctrees/language/extensions/canonical.doctree b/master/refman/.doctrees/language/extensions/canonical.doctree index 857a338c71..6152ad9b24 100644 Binary files a/master/refman/.doctrees/language/extensions/canonical.doctree and b/master/refman/.doctrees/language/extensions/canonical.doctree differ diff --git a/master/refman/.doctrees/language/extensions/evars.doctree b/master/refman/.doctrees/language/extensions/evars.doctree index e2fea27417..17bc68c209 100644 Binary files a/master/refman/.doctrees/language/extensions/evars.doctree and b/master/refman/.doctrees/language/extensions/evars.doctree differ diff --git a/master/refman/.doctrees/language/extensions/implicit-arguments.doctree b/master/refman/.doctrees/language/extensions/implicit-arguments.doctree index a68ec2f956..74313d8453 100644 Binary files a/master/refman/.doctrees/language/extensions/implicit-arguments.doctree and b/master/refman/.doctrees/language/extensions/implicit-arguments.doctree differ diff --git a/master/refman/.doctrees/language/extensions/match.doctree b/master/refman/.doctrees/language/extensions/match.doctree index 819b47c21c..5100cb3980 100644 Binary files a/master/refman/.doctrees/language/extensions/match.doctree and b/master/refman/.doctrees/language/extensions/match.doctree differ diff --git a/master/refman/.doctrees/proof-engine/ltac.doctree b/master/refman/.doctrees/proof-engine/ltac.doctree index 5dbc552571..1e6f681ef0 100644 Binary files a/master/refman/.doctrees/proof-engine/ltac.doctree and b/master/refman/.doctrees/proof-engine/ltac.doctree differ diff --git a/master/refman/.doctrees/proof-engine/ltac2.doctree b/master/refman/.doctrees/proof-engine/ltac2.doctree index c6319f98fb..843b3e0548 100644 Binary files a/master/refman/.doctrees/proof-engine/ltac2.doctree and b/master/refman/.doctrees/proof-engine/ltac2.doctree differ diff --git a/master/refman/.doctrees/proof-engine/ssreflect-proof-language.doctree b/master/refman/.doctrees/proof-engine/ssreflect-proof-language.doctree index ff185239f9..eea89e445b 100644 Binary files a/master/refman/.doctrees/proof-engine/ssreflect-proof-language.doctree and b/master/refman/.doctrees/proof-engine/ssreflect-proof-language.doctree differ diff --git a/master/refman/.doctrees/proof-engine/tactics.doctree b/master/refman/.doctrees/proof-engine/tactics.doctree index 2fcef3b372..c8747137ca 100644 Binary files a/master/refman/.doctrees/proof-engine/tactics.doctree and b/master/refman/.doctrees/proof-engine/tactics.doctree differ diff --git a/master/refman/.doctrees/proof-engine/vernacular-commands.doctree b/master/refman/.doctrees/proof-engine/vernacular-commands.doctree index 281a7c4cc1..fe1bfdba9d 100644 Binary files a/master/refman/.doctrees/proof-engine/vernacular-commands.doctree and b/master/refman/.doctrees/proof-engine/vernacular-commands.doctree differ diff --git a/master/refman/.doctrees/proofs/writing-proofs/equality.doctree b/master/refman/.doctrees/proofs/writing-proofs/equality.doctree index 3a28c0bef8..379f4a14d6 100644 Binary files a/master/refman/.doctrees/proofs/writing-proofs/equality.doctree and b/master/refman/.doctrees/proofs/writing-proofs/equality.doctree differ diff --git a/master/refman/.doctrees/proofs/writing-proofs/proof-mode.doctree b/master/refman/.doctrees/proofs/writing-proofs/proof-mode.doctree index 3cdb05c65a..3b52bb4fc1 100644 Binary files a/master/refman/.doctrees/proofs/writing-proofs/proof-mode.doctree and b/master/refman/.doctrees/proofs/writing-proofs/proof-mode.doctree differ diff --git a/master/refman/.doctrees/proofs/writing-proofs/reasoning-inductives.doctree b/master/refman/.doctrees/proofs/writing-proofs/reasoning-inductives.doctree index 1dff554f71..58f2074dcb 100644 Binary files a/master/refman/.doctrees/proofs/writing-proofs/reasoning-inductives.doctree and b/master/refman/.doctrees/proofs/writing-proofs/reasoning-inductives.doctree differ diff --git a/master/refman/.doctrees/user-extensions/syntax-extensions.doctree b/master/refman/.doctrees/user-extensions/syntax-extensions.doctree index 06ade9ef03..0609f30d24 100644 Binary files a/master/refman/.doctrees/user-extensions/syntax-extensions.doctree and b/master/refman/.doctrees/user-extensions/syntax-extensions.doctree differ diff --git a/master/refman/.doctrees/using/libraries/writing.doctree b/master/refman/.doctrees/using/libraries/writing.doctree index b5c9ccc742..e8edbccf2b 100644 Binary files a/master/refman/.doctrees/using/libraries/writing.doctree and b/master/refman/.doctrees/using/libraries/writing.doctree differ diff --git a/master/refman/language/extensions/match.html b/master/refman/language/extensions/match.html index c3ece0056a..f488c5bf4e 100644 --- a/master/refman/language/extensions/match.html +++ b/master/refman/language/extensions/match.html @@ -1563,13 +1563,13 @@

Printing of hidden subtermsPrint seq_rect.
seq_rect = fun (A : Type@{seq.u0}) (a : A) - (P : forall a0 : A, seq a a0 -> Type@{Top.68}) (f : P a (srefl a)) - (a0 : A) (s : seq a a0) => + (P : forall a0 : A, seq a a0 -> Type@{seq_rect.u0}) + (f : P a (srefl a)) (a0 : A) (s : seq a a0) => match s :> seq a a0 as s0 in (seq _ a1) return (P a1 s0) with | srefl _ => f end : forall (A : Type@{seq.u0}) (a : A) - (P : forall a0 : A, seq a a0 -> Type@{Top.68}), + (P : forall a0 : A, seq a a0 -> Type@{seq_rect.u0}), P a (srefl a) -> forall (a0 : A) (s : seq a a0), P a0 s Arguments seq_rect A%type_scope a P%function_scope f a0 s diff --git a/master/refman/proof-engine/ltac.html b/master/refman/proof-engine/ltac.html index ae6f3150ee..6974dee313 100644 --- a/master/refman/proof-engine/ltac.html +++ b/master/refman/proof-engine/ltac.html @@ -3375,7 +3375,7 @@

Timing a tactic that evaluates to a term: time_constrpose v.
Tactic evaluation (depth 1) ran for 0. secs (0.u,0.s) Tactic evaluation (depth 1) ran for 0. secs (0.u,0.s) -Tactic evaluation ran for 0. secs (0.u,0.s) +Tactic evaluation ran for 0.001 secs (0.001u,0.s) 1 goal n := 100 : nat @@ -4289,42 +4289,40 @@

Profiling L
No more goals.
Show Ltac Profile. -
total time: 1.172s +
total time: 2.079s tactic local total calls max ──────────────────────────────────────────┴──────┴──────┴───────┴─────────┘ -─tac ------------------------------------- 4.7% 100.0% 1 1.172s -─<Stdlib.Init.Tauto.with_uniform_flags> -- 0.0% 92.8% 26 0.128s -─<Stdlib.Init.Tauto.tauto_gen> ----------- 0.0% 92.7% 26 0.128s -─<Stdlib.Init.Tauto.tauto_intuitionistic> 0.0% 92.6% 26 0.128s -─t_tauto_intuit -------------------------- 0.1% 92.5% 26 0.128s -─<Stdlib.Init.Tauto.simplif> ------------- 57.0% 89.3% 26 0.126s -─<Stdlib.Init.Tauto.is_conj> ------------- 21.2% 21.2% 28756 0.005s -─elim id --------------------------------- 4.9% 4.9% 650 0.002s -─<Stdlib.Init.Tauto.is_disj> ------------- 3.7% 3.7% 1430 0.032s -─<Stdlib.Init.Tauto.axioms> -------------- 2.1% 3.1% 0 0.002s -─lia ------------------------------------- 0.1% 2.2% 28 0.012s +─tac ------------------------------------- 0.1% 100.0% 1 2.079s +─<Stdlib.Init.Tauto.with_uniform_flags> -- 0.0% 95.3% 26 0.180s +─<Stdlib.Init.Tauto.tauto_gen> ----------- 0.0% 95.3% 26 0.180s +─<Stdlib.Init.Tauto.tauto_intuitionistic> 0.0% 95.2% 26 0.180s +─t_tauto_intuit -------------------------- 0.1% 95.1% 26 0.180s +─<Stdlib.Init.Tauto.simplif> ------------- 61.3% 91.2% 26 0.177s +─<Stdlib.Init.Tauto.is_conj> ------------- 19.8% 19.8% 28756 0.013s +─elim id --------------------------------- 6.1% 6.1% 650 0.001s +─<Stdlib.Init.Tauto.axioms> -------------- 3.0% 3.9% 0 0.018s +─split ----------------------------------- 2.7% 2.7% 55 0.052s tactic local total calls max ────────────────────────────────────────────┴──────┴──────┴───────┴─────────┘ -─tac --------------------------------------- 4.7% 100.0% 1 1.172s - ├─<Stdlib.Init.Tauto.with_uniform_flags> -- 0.0% 92.7% 26 0.128s - │└<Stdlib.Init.Tauto.tauto_gen> ----------- 0.0% 92.7% 26 0.128s - │└<Stdlib.Init.Tauto.tauto_intuitionistic> 0.0% 92.6% 26 0.128s - │└t_tauto_intuit -------------------------- 0.1% 92.5% 26 0.128s - │ ├─<Stdlib.Init.Tauto.simplif> ----------- 57.0% 89.3% 26 0.126s - │ │ ├─<Stdlib.Init.Tauto.is_conj> --------- 21.2% 21.2% 28756 0.005s - │ │ ├─elim id ----------------------------- 4.9% 4.9% 650 0.002s - │ │ └─<Stdlib.Init.Tauto.is_disj> --------- 3.7% 3.7% 1430 0.032s - │ └─<Stdlib.Init.Tauto.axioms> ------------ 2.1% 3.1% 0 0.002s - └─lia ------------------------------------- 0.1% 2.2% 28 0.012s +─tac --------------------------------------- 0.1% 100.0% 1 2.079s + ├─<Stdlib.Init.Tauto.with_uniform_flags> -- 0.0% 95.3% 26 0.180s + │└<Stdlib.Init.Tauto.tauto_gen> ----------- 0.0% 95.2% 26 0.180s + │└<Stdlib.Init.Tauto.tauto_intuitionistic> 0.0% 95.2% 26 0.180s + │└t_tauto_intuit -------------------------- 0.1% 95.1% 26 0.180s + │ ├─<Stdlib.Init.Tauto.simplif> ----------- 61.3% 91.2% 26 0.177s + │ │ ├─<Stdlib.Init.Tauto.is_conj> --------- 19.8% 19.8% 28756 0.013s + │ │ └─elim id ----------------------------- 6.1% 6.1% 650 0.001s + │ └─<Stdlib.Init.Tauto.axioms> ------------ 3.0% 3.9% 0 0.018s + └─split ----------------------------------- 2.7% 2.7% 55 0.052s
Show Ltac Profile "lia". -
total time: 1.172s +
total time: 2.079s tactic local total calls max ───────┴──────┴──────┴───────┴─────────┘ -─lia -- 0.1% 2.2% 28 0.012s + tactic local total calls max ───────┴──────┴──────┴───────┴─────────┘ diff --git a/master/refman/proofs/writing-proofs/equality.html b/master/refman/proofs/writing-proofs/equality.html index d982d96fe3..ad8ebcfb9b 100644 --- a/master/refman/proofs/writing-proofs/equality.html +++ b/master/refman/proofs/writing-proofs/equality.html @@ -2636,7 +2636,7 @@

Computing in a term: eval and EvalTime assert (id (fact 8) = fact 8) by reflexivity. -
Finished transaction in 0.113 secs (0.102u,0.01s) (successful) +
Finished transaction in 0.175 secs (0.143u,0.032s) (successful) 1 goal H : id (fact 8) = fact 8 @@ -2644,7 +2644,7 @@

Computing in a term: eval and EvalTime assert (id (fact 9) = fact 9) by reflexivity. -
Finished transaction in 0.532 secs (0.532u,0.s) (successful) +
Finished transaction in 1.055 secs (1.055u,0.s) (successful) 1 goal H : id (fact 8) = fact 8 @@ -2707,7 +2707,7 @@

Computing in a term: eval and EvalTime assert (id (fact 100) = fact 100) by with_strategy -1 [id] abstract reflexivity. -
Finished transaction in 0.001 secs (0.001u,0.s) (successful) +
Finished transaction in 0.002 secs (0.002u,0.s) (successful) 1 goal H : id (fact 100) = fact 100 diff --git a/master/refman/searchindex.js b/master/refman/searchindex.js index 0c0fe005fb..141251c16b 100644 --- a/master/refman/searchindex.js +++ b/master/refman/searchindex.js @@ -1 +1 @@ -Search.setIndex({docnames:["addendum/canonical-structures","addendum/extended-pattern-matching","addendum/extraction","addendum/generalized-rewriting","addendum/implicit-coercions","addendum/micromega","addendum/miscellaneous-extensions","addendum/nsatz","addendum/parallel-proof-processing","addendum/program","addendum/rewrite-rules","addendum/ring","addendum/sprop","addendum/type-classes","addendum/universe-polymorphism","appendix/history-and-changes/index","appendix/indexes/index","changes","coq-attrindex","coq-cmdindex","coq-exnindex","coq-optindex","coq-tacindex","genindex","history","index","language/cic","language/coq-library","language/core/assumptions","language/core/basic","language/core/coinductive","language/core/conversion","language/core/definitions","language/core/index","language/core/inductive","language/core/modules","language/core/primitive","language/core/records","language/core/sections","language/core/sorts","language/core/variants","language/extensions/arguments-command","language/extensions/canonical","language/extensions/evars","language/extensions/implicit-arguments","language/extensions/index","language/extensions/match","language/gallina-extensions","language/gallina-specification-language","language/module-system","license","practical-tools/coq-commands","practical-tools/coqide","practical-tools/utilities","proof-engine/ltac","proof-engine/ltac2","proof-engine/proof-handling","proof-engine/ssreflect-proof-language","proof-engine/tactics","proof-engine/vernacular-commands","proofs/automatic-tactics/auto","proofs/automatic-tactics/index","proofs/automatic-tactics/logic","proofs/creating-tactics/index","proofs/writing-proofs/equality","proofs/writing-proofs/index","proofs/writing-proofs/proof-mode","proofs/writing-proofs/reasoning-inductives","proofs/writing-proofs/rewriting","std-glossindex","user-extensions/proof-schemes","user-extensions/syntax-extensions","using/libraries/funind","using/libraries/index","using/libraries/writing","using/tools/coqdoc","using/tools/index","zebibliography"],envversion:{"coqrst.coqdomain":2,"sphinx.domains.c":2,"sphinx.domains.changeset":1,"sphinx.domains.citation":1,"sphinx.domains.cpp":5,"sphinx.domains.index":1,"sphinx.domains.javascript":2,"sphinx.domains.math":2,"sphinx.domains.python":3,"sphinx.domains.rst":2,"sphinx.domains.std":2,"sphinx.ext.todo":2,sphinx:56},filenames:["addendum/canonical-structures.rst","addendum/extended-pattern-matching.rst","addendum/extraction.rst","addendum/generalized-rewriting.rst","addendum/implicit-coercions.rst","addendum/micromega.rst","addendum/miscellaneous-extensions.rst","addendum/nsatz.rst","addendum/parallel-proof-processing.rst","addendum/program.rst","addendum/rewrite-rules.rst","addendum/ring.rst","addendum/sprop.rst","addendum/type-classes.rst","addendum/universe-polymorphism.rst","appendix/history-and-changes/index.rst","appendix/indexes/index.rst","changes.rst","coq-attrindex.rst","coq-cmdindex.rst","coq-exnindex.rst","coq-optindex.rst","coq-tacindex.rst","genindex.rst","history.rst","index.rst","language/cic.rst","language/coq-library.rst","language/core/assumptions.rst","language/core/basic.rst","language/core/coinductive.rst","language/core/conversion.rst","language/core/definitions.rst","language/core/index.rst","language/core/inductive.rst","language/core/modules.rst","language/core/primitive.rst","language/core/records.rst","language/core/sections.rst","language/core/sorts.rst","language/core/variants.rst","language/extensions/arguments-command.rst","language/extensions/canonical.rst","language/extensions/evars.rst","language/extensions/implicit-arguments.rst","language/extensions/index.rst","language/extensions/match.rst","language/gallina-extensions.rst","language/gallina-specification-language.rst","language/module-system.rst","license.rst","practical-tools/coq-commands.rst","practical-tools/coqide.rst","practical-tools/utilities.rst","proof-engine/ltac.rst","proof-engine/ltac2.rst","proof-engine/proof-handling.rst","proof-engine/ssreflect-proof-language.rst","proof-engine/tactics.rst","proof-engine/vernacular-commands.rst","proofs/automatic-tactics/auto.rst","proofs/automatic-tactics/index.rst","proofs/automatic-tactics/logic.rst","proofs/creating-tactics/index.rst","proofs/writing-proofs/equality.rst","proofs/writing-proofs/index.rst","proofs/writing-proofs/proof-mode.rst","proofs/writing-proofs/reasoning-inductives.rst","proofs/writing-proofs/rewriting.rst","std-glossindex.rst","user-extensions/proof-schemes.rst","user-extensions/syntax-extensions.rst","using/libraries/funind.rst","using/libraries/index.rst","using/libraries/writing.rst","using/tools/coqdoc.rst","using/tools/index.rst","zebibliography.rst"],objects:{"":[[71,0,1,"coq:exn.'via'-and-'abstract'-cannot-be-used-together","'via' and 'abstract' cannot be used together"],[54,1,1,"coq:tacn.+-(backtracking-branching)","+ (backtracking branching)"],[57,1,1,"coq:tacn.=>","=>"],[66,3,1,"coq:cmd.Abort","Abort"],[59,3,1,"coq:cmd.About","About"],[71,2,1,"coq:warn.Activation-of-abbreviations-does-not-expect-mentioning-a-grammar-entry","Activation of abbreviations does not expect mentioning a grammar entry"],[71,2,1,"coq:warn.Activation-of-abbreviations-does-not-expect-mentioning-a-scope","Activation of abbreviations does not expect mentioning a scope"],[29,3,1,"coq:cmd.Add","Add"],[11,3,1,"coq:cmd.Add-Field","Add Field"],[3,3,1,"coq:cmd.Add-Morphism","Add Morphism"],[3,3,1,"coq:cmd.Add-Parametric-Morphism","Add Parametric Morphism"],[3,3,1,"coq:cmd.Add-Parametric-Relation","Add Parametric Relation"],[3,3,1,"coq:cmd.Add-Parametric-Setoid","Add Parametric Setoid"],[3,3,1,"coq:cmd.Add-Relation","Add Relation"],[11,3,1,"coq:cmd.Add-Ring","Add Ring"],[3,3,1,"coq:cmd.Add-Setoid","Add Setoid"],[5,3,1,"coq:cmd.Add-Zify","Add Zify"],[9,3,1,"coq:cmd.Admit-Obligations","Admit Obligations"],[66,3,1,"coq:cmd.Admitted","Admitted"],[12,4,1,"coq:flag.Allow-StrictProp","Allow StrictProp"],[44,0,1,"coq:exn.Argument-at-position-\u2018natural\u2019-is-mentioned-more-than-once","Argument at position \u2018natural\u2019 is mentioned more than once"],[54,0,1,"coq:exn.Argument-of-match-does-not-evaluate-to-a-term","Argument of match does not evaluate to a term"],[41,3,1,"coq:cmd.Arguments","Arguments"],[44,0,1,"coq:exn.Arguments-given-by-name-or-position-not-supported-in-explicit-mode","Arguments given by name or position not supported in explicit mode"],[11,0,1,"coq:exn.Arguments-of-ring_simplify-do-not-have-all-the-same-type","Arguments of ring_simplify do not have all the same type"],[41,0,1,"coq:exn.Arguments-of-section-variables-such-as-\u2018name\u2019-may-not-be-renamed","Arguments of section variables such as \u2018name\u2019 may not be renamed"],[46,4,1,"coq:flag.Asymmetric-Patterns","Asymmetric Patterns"],[66,0,1,"coq:exn.Attempt-to-save-an-incomplete-proof","Attempt to save an incomplete proof"],[29,3,1,"coq:cmd.Attributes","Attributes"],[34,4,1,"coq:flag.Auto-Template-Polymorphism","Auto Template Polymorphism"],[34,4,1,"coq:flag.Automatic-Proposition-Inductives","Automatic Proposition Inductives"],[34,2,1,"coq:warn.Automatically-declaring-\u2018ident\u2019-as-template-polymorphic","Automatically declaring \u2018ident\u2019 as template polymorphic"],[28,3,1,"coq:cmd.Axiom","Axiom"],[28,3,1,"coq:cmd.Axioms","Axioms"],[59,3,1,"coq:cmd.Back","Back"],[59,3,1,"coq:cmd.BackTo","BackTo"],[11,0,1,"coq:exn.Bad-lemma-for-decidability-of-equality","Bad lemma for decidability of equality"],[59,0,1,"coq:exn.Bad-magic-number","Bad magic number"],[64,0,1,"coq:exn.Bad-occurrence-number-of-\u2018qualid\u2019","Bad occurrence number of \u2018qualid\u2019"],[12,2,1,"coq:warn.Bad-relevance","Bad relevance"],[11,0,1,"coq:exn.Bad-ring-structure","Bad ring structure"],[71,3,1,"coq:cmd.Bind-Scope","Bind Scope"],[67,4,1,"coq:flag.Boolean-Equality-Schemes","Boolean Equality Schemes"],[5,5,1,"coq:thm.Bound-on-the-ceiling-function","Bound on the ceiling function"],[66,0,1,"coq:exn.Brackets-do-not-support-multi-goal-selectors","Brackets do not support multi-goal selectors"],[66,6,1,"coq:opt.Bullet-Behavior","Bullet Behavior"],[72,2,1,"coq:warn.Cannot-build-functional-inversion-principle","Cannot build functional inversion principle"],[58,0,1,"coq:exn.Cannot-change-\u2018ident\u2019,-it-is-used-in-conclusion","Cannot change \u2018ident\u2019, it is used in conclusion"],[58,0,1,"coq:exn.Cannot-change-\u2018ident\u2019,-it-is-used-in-hypothesis-\u2018ident\u2019","Cannot change \u2018ident\u2019, it is used in hypothesis \u2018ident\u2019"],[60,0,1,"coq:exn.Cannot-coerce-\u2018qualid\u2019-to-an-evaluable-reference","Cannot coerce \u2018qualid\u2019 to an evaluable reference"],[72,2,1,"coq:warn.Cannot-define-graph-for-\u2018ident\u2019","Cannot define graph for \u2018ident\u2019"],[72,2,1,"coq:warn.Cannot-define-principle(s)-for-\u2018ident\u2019","Cannot define principle(s) for \u2018ident\u2019"],[11,0,1,"coq:exn.Cannot-find-a-declared-ring-structure-for-equality-\u2018term\u2019","Cannot find a declared ring structure for equality \u2018term\u2019"],[11,0,1,"coq:exn.Cannot-find-a-declared-ring-structure-over-\u2018term\u2019","Cannot find a declared ring structure over \u2018term\u2019"],[64,0,1,"coq:exn.Cannot-find-a-relation-to-rewrite","Cannot find a relation to rewrite"],[64,0,1,"coq:exn.Cannot-find-any-non-recursive-equality-over-\u2018ident\u2019","Cannot find any non-recursive equality over \u2018ident\u2019"],[72,0,1,"coq:exn.Cannot-find-induction-information-on-\u2018qualid\u2019","Cannot find induction information on \u2018qualid\u2019"],[72,0,1,"coq:exn.Cannot-find-inversion-information-for-hypothesis-\u2018ident\u2019","Cannot find inversion information for hypothesis \u2018ident\u2019"],[59,0,1,"coq:exn.Cannot-find-library-foo-in-loadpath","Cannot find library foo in loadpath"],[4,0,1,"coq:exn.Cannot-find-the-source-class-of-\u2018qualid\u2019","Cannot find the source class of \u2018qualid\u2019"],[4,0,1,"coq:exn.Cannot-find-the-target-class","Cannot find the target class"],[35,2,1,"coq:warn.Cannot-import-local-constant,-it-will-be-ignored","Cannot import local constant, it will be ignored"],[71,0,1,"coq:exn.Cannot-interpret-in-\u2018scope_name\u2019-because-\u2018qualid\u2019-could-not-be-found-in-the-current-environment","Cannot interpret in \u2018scope_name\u2019 because \u2018qualid\u2019 could not be found in the current environment"],[71,0,1,"coq:exn.Cannot-interpret-this-number-as-a-value-of-type-\u2018type\u2019","Cannot interpret this number as a value of type \u2018type\u2019"],[71,0,1,"coq:exn.Cannot-interpret-this-string-as-a-value-of-type-\u2018type\u2019","Cannot interpret this string as a value of type \u2018type\u2019"],[59,0,1,"coq:exn.Cannot-load-\u2018qualid\u2019:-no-physical-path-bound-to-\u2018dirpath\u2019","Cannot load \u2018qualid\u2019: no physical path bound to \u2018dirpath\u2019"],[58,0,1,"coq:exn.Cannot-move-\u2018ident\u2019-after-\u2018ident\u2019:-it-depends-on-\u2018ident\u2019","Cannot move \u2018ident\u2019 after \u2018ident\u2019: it depends on \u2018ident\u2019"],[58,0,1,"coq:exn.Cannot-move-\u2018ident\u2019-after-\u2018ident\u2019:-it-occurs-in-the-type-of-\u2018ident\u2019","Cannot move \u2018ident\u2019 after \u2018ident\u2019: it occurs in the type of \u2018ident\u2019"],[62,0,1,"coq:exn.Cannot-recognize-a-boolean-equality","Cannot recognize a boolean equality"],[67,0,1,"coq:exn.Cannot-recognize-a-statement-based-on-\u2018reference\u2019","Cannot recognize a statement based on \u2018reference\u2019"],[4,0,1,"coq:exn.Cannot-recognize-\u2018coercion_class\u2019-as-a-source-class-of-\u2018qualid\u2019","Cannot recognize \u2018coercion_class\u2019 as a source class of \u2018qualid\u2019"],[64,0,1,"coq:exn.Cannot-turn-[inductive|constructor]-into-an-evaluable-reference","Cannot turn [inductive|constructor] into an evaluable reference"],[72,0,1,"coq:exn.Cannot-use-mutual-definition-with-well-founded-recursion-or-measure","Cannot use mutual definition with well-founded recursion or measure"],[42,3,1,"coq:cmd.Canonical-Structure","Canonical Structure"],[59,0,1,"coq:exn.Can\u2019t-find-file-\u2018ident\u2019-on-loadpath","Can\u2019t find file \u2018ident\u2019 on loadpath"],[67,4,1,"coq:flag.Case-Analysis-Schemes","Case Analysis Schemes"],[5,5,1,"coq:thm.Case-split","Case split"],[40,0,1,"coq:exn.Casts-are-not-supported-in-this-pattern","Casts are not supported in this pattern"],[2,3,1,"coq:cmd.Cd","Cd"],[59,3,1,"coq:cmd.Check","Check"],[13,3,1,"coq:cmd.Class","Class"],[71,3,1,"coq:cmd.Close-Scope","Close Scope"],[30,3,1,"coq:cmd.CoFixpoint","CoFixpoint"],[30,3,1,"coq:cmd.CoInductive","CoInductive"],[4,3,1,"coq:cmd.Coercion","Coercion"],[66,3,1,"coq:cmd.Collection","Collection"],[67,3,1,"coq:cmd.Combined-Scheme","Combined Scheme"],[29,3,1,"coq:cmd.Comments","Comments"],[64,3,1,"coq:cmd.Compute","Compute"],[54,0,1,"coq:exn.Condition-not-satisfied","Condition not satisfied"],[28,3,1,"coq:cmd.Conjecture","Conjecture"],[28,3,1,"coq:cmd.Conjectures","Conjectures"],[14,3,1,"coq:cmd.Constraint","Constraint"],[38,3,1,"coq:cmd.Context","Context"],[44,4,1,"coq:flag.Contextual-Implicit","Contextual Implicit"],[51,4,1,"coq:flag.Coqtop-Exit-On-Error","Coqtop Exit On Error"],[32,3,1,"coq:cmd.Corollary","Corollary"],[60,3,1,"coq:cmd.Create-HintDb","Create HintDb"],[14,7,1,"coq:attr.Cumulative","Cumulative"],[14,4,1,"coq:flag.Cumulativity-Weak-Constraints","Cumulativity Weak Constraints"],[54,3,1,"coq:cmd.Debug","Debug"],[59,6,1,"coq:opt.Debug","Debug"],[60,4,1,"coq:flag.Debug-Auto","Debug Auto"],[60,4,1,"coq:flag.Debug-Eauto","Debug Eauto"],[57,4,1,"coq:flag.Debug-SsrMatching","Debug SsrMatching"],[57,4,1,"coq:flag.Debug-Ssreflect","Debug Ssreflect"],[60,4,1,"coq:flag.Debug-Trivial","Debug Trivial"],[54,0,1,"coq:exn.Debug-mode-not-available-in-the-IDE","Debug mode not available in the IDE"],[67,4,1,"coq:flag.Decidable-Equality-Schemes","Decidable Equality Schemes"],[71,3,1,"coq:cmd.Declare-Custom-Entry","Declare Custom Entry"],[64,3,1,"coq:cmd.Declare-Equivalent-Keys","Declare Equivalent Keys"],[13,3,1,"coq:cmd.Declare-Instance","Declare Instance"],[64,3,1,"coq:cmd.Declare-Left-Step","Declare Left Step"],[59,3,1,"coq:cmd.Declare-ML-Module","Declare ML Module"],[35,3,1,"coq:cmd.Declare-Module","Declare Module"],[3,3,1,"coq:cmd.Declare-Morphism","Declare Morphism"],[64,3,1,"coq:cmd.Declare-Reduction","Declare Reduction"],[64,3,1,"coq:cmd.Declare-Right-Step","Declare Right Step"],[71,3,1,"coq:cmd.Declare-Scope","Declare Scope"],[60,2,1,"coq:warn.Declaring-arbitrary-terms-as-hints-is-fragile-and-deprecated;-it-is-recommended-to-declare-a-toplevel-constant-instead","Declaring arbitrary terms as hints is fragile and deprecated; it is recommended to declare a toplevel constant instead"],[58,6,1,"coq:opt.Default-Goal-Selector","Default Goal Selector"],[66,6,1,"coq:opt.Default-Proof-Mode","Default Proof Mode"],[66,6,1,"coq:opt.Default-Proof-Using","Default Proof Using"],[59,6,1,"coq:opt.Default-Timeout","Default Timeout"],[66,3,1,"coq:cmd.Defined","Defined"],[32,3,1,"coq:cmd.Definition","Definition"],[12,4,1,"coq:flag.Definitional-UIP","Definitional UIP"],[71,3,1,"coq:cmd.Delimit-Scope","Delimit Scope"],[34,4,1,"coq:flag.Dependent-Proposition-Eliminators","Dependent Proposition Eliminators"],[6,3,1,"coq:cmd.Derive","Derive"],[67,3,1,"coq:cmd.Derive-Dependent-Inversion","Derive Dependent Inversion"],[67,3,1,"coq:cmd.Derive-Dependent-Inversion_clear","Derive Dependent Inversion_clear"],[67,3,1,"coq:cmd.Derive-Inversion","Derive Inversion"],[67,3,1,"coq:cmd.Derive-Inversion_clear","Derive Inversion_clear"],[66,6,1,"coq:opt.Diffs","Diffs"],[71,3,1,"coq:cmd.Disable-Notation","Disable Notation"],[59,3,1,"coq:cmd.Drop","Drop"],[5,6,1,"coq:opt.Dump-Arith","Dump Arith"],[59,0,1,"coq:exn.Dynlink-error:-execution-of-module-initializers-in-the","Dynlink error: execution of module initializers in the"],[46,0,1,"coq:exn.Either-there-is-a-type-incompatibility-or-the-problem-involves-dependencies","Either there is a type incompatibility or the problem involves dependencies"],[67,4,1,"coq:flag.Elimination-Schemes","Elimination Schemes"],[71,3,1,"coq:cmd.Enable-Notation","Enable Notation"],[38,3,1,"coq:cmd.End","End"],[71,0,1,"coq:exn.End-of-quoted-string-not-followed-by-a-space-in-notation","End of quoted string not followed by a space in notation"],[64,3,1,"coq:cmd.Eval","Eval"],[32,3,1,"coq:cmd.Example","Example"],[13,3,1,"coq:cmd.Existing-Class","Existing Class"],[13,3,1,"coq:cmd.Existing-Instance","Existing Instance"],[13,3,1,"coq:cmd.Existing-Instances","Existing Instances"],[35,3,1,"coq:cmd.Export","Export"],[54,0,1,"coq:exn.Expression-does-not-evaluate-to-a-tactic","Expression does not evaluate to a tactic"],[2,3,1,"coq:cmd.Extract-Callback","Extract Callback"],[2,0,1,"coq:exn.Extract-Callback-is-supported-only-for-OCaml-extraction","Extract Callback is supported only for OCaml extraction"],[2,3,1,"coq:cmd.Extract-Constant","Extract Constant"],[2,3,1,"coq:cmd.Extract-Foreign-Constant","Extract Foreign Constant"],[2,0,1,"coq:exn.Extract-Foreign-Constant-is-supported-only-for-OCaml-extraction","Extract Foreign Constant is supported only for OCaml extraction"],[2,0,1,"coq:exn.Extract-Foreign-Constant-is-supported-only-for-functions","Extract Foreign Constant is supported only for functions"],[2,3,1,"coq:cmd.Extract-Inductive","Extract Inductive"],[2,3,1,"coq:cmd.Extract-Inlined-Constant","Extract Inlined Constant"],[2,3,1,"coq:cmd.Extraction","Extraction"],[2,4,1,"coq:flag.Extraction-AutoInline","Extraction AutoInline"],[2,3,1,"coq:cmd.Extraction-Blacklist","Extraction Blacklist"],[2,4,1,"coq:flag.Extraction-Conservative-Types","Extraction Conservative Types"],[2,6,1,"coq:opt.Extraction-File-Comment","Extraction File Comment"],[2,6,1,"coq:opt.Extraction-Flag","Extraction Flag"],[2,3,1,"coq:cmd.Extraction-Implicit","Extraction Implicit"],[2,3,1,"coq:cmd.Extraction-Inline","Extraction Inline"],[2,4,1,"coq:flag.Extraction-KeepSingleton","Extraction KeepSingleton"],[2,3,1,"coq:cmd.Extraction-Language","Extraction Language"],[2,3,1,"coq:cmd.Extraction-Library","Extraction Library"],[2,3,1,"coq:cmd.Extraction-NoInline","Extraction NoInline"],[2,4,1,"coq:flag.Extraction-Optimize","Extraction Optimize"],[2,6,1,"coq:opt.Extraction-Output-Directory","Extraction Output Directory"],[2,4,1,"coq:flag.Extraction-SafeImplicits","Extraction SafeImplicits"],[2,3,1,"coq:cmd.Extraction-TestCompile","Extraction TestCompile"],[2,4,1,"coq:flag.Extraction-TypeExpand","Extraction TypeExpand"],[32,3,1,"coq:cmd.Fact","Fact"],[59,3,1,"coq:cmd.Fail","Fail"],[54,0,1,"coq:exn.Failed-to-progress","Failed to progress"],[59,4,1,"coq:flag.Fast-Name-Printing","Fast Name Printing"],[59,0,1,"coq:exn.File-not-found-on-loadpath:-\u2018string\u2019","File not found on loadpath: \u2018string\u2019"],[59,0,1,"coq:exn.Files-processed-by-Load-cannot-leave-open-proofs","Files processed by Load cannot leave open proofs"],[9,3,1,"coq:cmd.Final-Obligation","Final Obligation"],[62,6,1,"coq:opt.Firstorder-Depth","Firstorder Depth"],[62,6,1,"coq:opt.Firstorder-Solver","Firstorder Solver"],[34,3,1,"coq:cmd.Fixpoint","Fixpoint"],[41,0,1,"coq:exn.Flag-'rename'-expected-to-rename-\u2018name\u2019-into-\u2018name\u2019","Flag 'rename' expected to rename \u2018name\u2019 into \u2018name\u2019"],[66,3,1,"coq:cmd.Focus","Focus"],[46,0,1,"coq:exn.Found-a-constructor-of-inductive-type-term-while-a-constructor-of-term-is-expected","Found a constructor of inductive type term while a constructor of term is expected"],[64,0,1,"coq:exn.Found-an-\"at\"-clause-without-\"with\"-clause","Found an "at" clause without "with" clause"],[71,2,1,"coq:warn.Found-no-matching-notation-to-enable-or-disable","Found no matching notation to enable or disable"],[64,0,1,"coq:exn.Found-no-subterm-matching-\u2018term\u2019-in-the-current-goal","Found no subterm matching \u2018term\u2019 in the current goal"],[64,0,1,"coq:exn.Found-no-subterm-matching-\u2018term\u2019-in-\u2018ident\u2019","Found no subterm matching \u2018term\u2019 in \u2018ident\u2019"],[4,0,1,"coq:exn.Found-target-class-\u2018coercion_class\u2019-instead-of-\u2018coercion_class\u2019","Found target class \u2018coercion_class\u2019 instead of \u2018coercion_class\u2019"],[59,3,1,"coq:cmd.From-\u2026-Dependency","From \u2026 Dependency"],[59,3,1,"coq:cmd.From-\u2026-Require","From \u2026 Require"],[4,0,1,"coq:exn.Funclass-cannot-be-a-source-class","Funclass cannot be a source class"],[72,3,1,"coq:cmd.Function","Function"],[72,3,1,"coq:cmd.Functional-Case","Functional Case"],[72,3,1,"coq:cmd.Functional-Scheme","Functional Scheme"],[44,3,1,"coq:cmd.Generalizable","Generalizable"],[72,3,1,"coq:cmd.Generate-graph-for","Generate graph for"],[66,3,1,"coq:cmd.Goal","Goal"],[59,4,1,"coq:flag.Guard-Checking","Guard Checking"],[66,3,1,"coq:cmd.Guarded","Guarded"],[60,3,1,"coq:cmd.Hint-Constants","Hint Constants"],[60,3,1,"coq:cmd.Hint-Constructors","Hint Constructors"],[60,3,1,"coq:cmd.Hint-Cut","Hint Cut"],[60,3,1,"coq:cmd.Hint-Extern","Hint Extern"],[60,3,1,"coq:cmd.Hint-Immediate","Hint Immediate"],[60,3,1,"coq:cmd.Hint-Mode","Hint Mode"],[60,3,1,"coq:cmd.Hint-Opaque","Hint Opaque"],[60,3,1,"coq:cmd.Hint-Projections","Hint Projections"],[60,3,1,"coq:cmd.Hint-Resolve","Hint Resolve"],[60,3,1,"coq:cmd.Hint-Rewrite","Hint Rewrite"],[60,3,1,"coq:cmd.Hint-Transparent","Hint Transparent"],[60,3,1,"coq:cmd.Hint-Unfold","Hint Unfold"],[60,3,1,"coq:cmd.Hint-Variables","Hint Variables"],[57,3,1,"coq:cmd.Hint-View-for","Hint View for"],[57,3,1,"coq:cmd.Hint-View-for-apply","Hint View for apply"],[57,3,1,"coq:cmd.Hint-View-for-move","Hint View for move"],[28,3,1,"coq:cmd.Hypotheses","Hypotheses"],[28,3,1,"coq:cmd.Hypothesis","Hypothesis"],[72,0,1,"coq:exn.Hypothesis-\u2018ident\u2019-must-contain-at-least-one-Function","Hypothesis \u2018ident\u2019 must contain at least one Function"],[66,6,1,"coq:opt.Hyps-Limit","Hyps Limit"],[62,0,1,"coq:exn.I-don\u2019t-know-how-to-handle-dependent-equality","I don\u2019t know how to handle dependent equality"],[4,3,1,"coq:cmd.Identity-Coercion","Identity Coercion"],[13,2,1,"coq:warn.Ignored-instance-declaration-for-\u201c\u2018ident\u2019\u201d:-\u201c\u2018term\u2019\u201d-is-not-a-class","Ignored instance declaration for \u201c\u2018ident\u2019\u201d: \u201c\u2018term\u2019\u201d is not a class"],[44,2,1,"coq:warn.Ignoring-implicit-binder-declaration-in-unexpected-position","Ignoring implicit binder declaration in unexpected position"],[9,0,1,"coq:exn.Ill-formed-recursive-definition","Ill-formed recursive definition"],[34,0,1,"coq:exn.Ill-formed-template-inductive-declaration:-not-polymorphic-on-any-universe","Ill-formed template inductive declaration: not polymorphic on any universe"],[44,4,1,"coq:flag.Implicit-Arguments","Implicit Arguments"],[44,3,1,"coq:cmd.Implicit-Type","Implicit Type"],[44,3,1,"coq:cmd.Implicit-Types","Implicit Types"],[35,3,1,"coq:cmd.Import","Import"],[35,3,1,"coq:cmd.Include","Include"],[35,3,1,"coq:cmd.Include-Type","Include Type"],[57,0,1,"coq:exn.Incorrect-number-of-tactics-(expected-N-tactics,-was-given-M)","Incorrect number of tactics (expected N tactics, was given M)"],[34,3,1,"coq:cmd.Inductive","Inductive"],[71,3,1,"coq:cmd.Infix","Infix"],[54,3,1,"coq:cmd.Info","Info"],[60,4,1,"coq:flag.Info-Auto","Info Auto"],[60,4,1,"coq:flag.Info-Eauto","Info Eauto"],[54,6,1,"coq:opt.Info-Level","Info Level"],[5,4,1,"coq:flag.Info-Micromega","Info Micromega"],[60,4,1,"coq:flag.Info-Trivial","Info Trivial"],[59,3,1,"coq:cmd.Inspect","Inspect"],[13,3,1,"coq:cmd.Instance","Instance"],[59,3,1,"coq:cmd.Instructions","Instructions"],[62,4,1,"coq:flag.Intuition-Negation-Unfolding","Intuition Negation Unfolding"],[59,0,1,"coq:exn.Invalid-backtrack","Invalid backtrack"],[67,8,1,"coq:table.Keep-Equalities","Keep Equalities"],[67,4,1,"coq:flag.Keep-Proof-Equalities","Keep Proof Equalities"],[64,4,1,"coq:flag.Kernel-Term-Sharing","Kernel Term Sharing"],[64,4,1,"coq:flag.Keyed-Unification","Keyed Unification"],[38,0,1,"coq:exn.Last-block-to-end-has-name-\u2018ident\u2019","Last block to end has name \u2018ident\u2019"],[32,3,1,"coq:cmd.Lemma","Lemma"],[38,3,1,"coq:cmd.Let","Let"],[38,3,1,"coq:cmd.Let-CoFixpoint","Let CoFixpoint"],[38,3,1,"coq:cmd.Let-Fixpoint","Let Fixpoint"],[5,4,1,"coq:flag.Lia-Cache","Lia Cache"],[59,3,1,"coq:cmd.Load","Load"],[59,0,1,"coq:exn.Load-is-not-supported-inside-proofs","Load is not supported inside proofs"],[59,3,1,"coq:cmd.Locate","Locate"],[59,3,1,"coq:cmd.Locate-File","Locate File"],[59,3,1,"coq:cmd.Locate-Library","Locate Library"],[59,3,1,"coq:cmd.Locate-Ltac","Locate Ltac"],[59,3,1,"coq:cmd.Locate-Ltac2","Locate Ltac2"],[59,3,1,"coq:cmd.Locate-Module","Locate Module"],[59,3,1,"coq:cmd.Locate-Term","Locate Term"],[60,6,1,"coq:opt.Loose-Hint-Behavior","Loose Hint Behavior"],[54,3,1,"coq:cmd.Ltac","Ltac"],[54,4,1,"coq:flag.Ltac-Backtrace","Ltac Backtrace"],[54,4,1,"coq:flag.Ltac-Batch-Debug","Ltac Batch Debug"],[54,4,1,"coq:flag.Ltac-Debug","Ltac Debug"],[54,4,1,"coq:flag.Ltac-Profiling","Ltac Profiling"],[55,3,1,"coq:cmd.Ltac2","Ltac2"],[55,4,1,"coq:flag.Ltac2-Backtrace","Ltac2 Backtrace"],[55,3,1,"coq:cmd.Ltac2-Check","Ltac2 Check"],[55,3,1,"coq:cmd.Ltac2-Eval","Ltac2 Eval"],[55,3,1,"coq:cmd.Ltac2-Globalize","Ltac2 Globalize"],[55,4,1,"coq:flag.Ltac2-In-Ltac1-Profiling","Ltac2 In Ltac1 Profiling"],[55,3,1,"coq:cmd.Ltac2-Notation","Ltac2 Notation"],[55,3,1,"coq:cmd.Ltac2-Notation-(abbreviation)","Ltac2 Notation (abbreviation)"],[55,3,1,"coq:cmd.Ltac2-Set","Ltac2 Set"],[55,3,1,"coq:cmd.Ltac2-Type","Ltac2 Type"],[55,4,1,"coq:flag.Ltac2-Typed-Notations","Ltac2 Typed Notations"],[55,3,1,"coq:cmd.Ltac2-external","Ltac2 external"],[44,2,1,"coq:warn.Making-shadowed-name-of-implicit-argument-accessible-by-position","Making shadowed name of implicit argument accessible by position"],[66,4,1,"coq:flag.Mangle-Names","Mangle Names"],[66,4,1,"coq:flag.Mangle-Names-Light","Mangle Names Light"],[66,6,1,"coq:opt.Mangle-Names-Prefix","Mangle Names Prefix"],[44,4,1,"coq:flag.Maximal-Implicit-Insertion","Maximal Implicit Insertion"],[71,0,1,"coq:exn.Missing-mapping-for-constructor-\u2018qualid\u2019","Missing mapping for constructor \u2018qualid\u2019"],[35,3,1,"coq:cmd.Module","Module"],[35,3,1,"coq:cmd.Module-Type","Module Type"],[59,0,1,"coq:exn.Module/section-\u2018qualid\u2019-not-found","Module/section \u2018qualid\u2019 not found"],[14,7,1,"coq:attr.Monomorphic","Monomorphic"],[71,0,1,"coq:exn.More-than-one-interpretation-bound-to-this-notation,-confirm-with-the-\"all\"-modifier","More than one interpretation bound to this notation, confirm with the "all" modifier"],[71,0,1,"coq:exn.Multiple-'via'-options","Multiple 'via' options"],[71,0,1,"coq:exn.Multiple-'warning-after'-or-'abstract-after'-options","Multiple 'warning after' or 'abstract after' options"],[64,6,1,"coq:opt.NativeCompute-Profile-Filename","NativeCompute Profile Filename"],[64,4,1,"coq:flag.NativeCompute-Profiling","NativeCompute Profiling"],[64,4,1,"coq:flag.NativeCompute-Timing","NativeCompute Timing"],[66,4,1,"coq:flag.Nested-Proofs-Allowed","Nested Proofs Allowed"],[66,2,1,"coq:warn.New-Collection-definition-of-\u2018ident\u2019-shadows-the-previous-one","New Collection definition of \u2018ident\u2019 shadows the previous one"],[9,3,1,"coq:cmd.Next-Obligation","Next Obligation"],[5,4,1,"coq:flag.Nia-Cache","Nia Cache"],[54,0,1,"coq:exn.No-applicable-tactic","No applicable tactic"],[72,0,1,"coq:exn.No-argument-name-\u2018ident\u2019","No argument name \u2018ident\u2019"],[54,0,1,"coq:exn.No-evars","No evars"],[35,0,1,"coq:exn.No-field-named-\u2018ident\u2019-in-\u2018qualid\u2019","No field named \u2018ident\u2019 in \u2018qualid\u2019"],[66,0,1,"coq:exn.No-focused-proof","No focused proof"],[66,0,1,"coq:exn.No-focused-proof-(No-proof-editing-in-progress)","No focused proof (No proof-editing in progress)"],[66,0,1,"coq:exn.No-focused-proof-to-restart","No focused proof to restart"],[64,0,1,"coq:exn.No-head-constant-to-reduce","No head constant to reduce"],[54,0,1,"coq:exn.No-matching-clauses-for-match","No matching clauses for match"],[54,0,1,"coq:exn.No-matching-clauses-for-match-goal","No matching clauses for match goal"],[71,0,1,"coq:exn.No-notation-provided","No notation provided"],[67,0,1,"coq:exn.No-primitive-equality-found","No primitive equality found"],[58,0,1,"coq:exn.No-product-even-after-head-reduction","No product even after head-reduction"],[3,0,1,"coq:exn.No-progress-made","No progress made"],[58,0,1,"coq:exn.No-quantified-hypothesis-named-\u2018ident\u2019-in-current-goal-even-after-head-reduction","No quantified hypothesis named \u2018ident\u2019 in current goal even after head-reduction"],[58,0,1,"coq:exn.No-such-assumption","No such assumption"],[58,0,1,"coq:exn.No-such-binder","No such binder"],[58,0,1,"coq:exn.No-such-bound-variable-\u2018ident\u2019-(no-bound-variables-at-all-in-the-expression)","No such bound variable \u2018ident\u2019 (no bound variables at all in the expression)"],[66,0,1,"coq:exn.No-such-goal","No such goal"],[66,0,1,"coq:exn.No-such-goal-(\u2018ident\u2019)","No such goal (\u2018ident\u2019)"],[66,0,1,"coq:exn.No-such-goal-(\u2018natural\u2019)","No such goal (\u2018natural\u2019)"],[58,0,1,"coq:exn.No-such-hypothesis:-\u2018ident\u2019","No such hypothesis: \u2018ident\u2019"],[58,0,1,"coq:exn.No-\u2018natural\u2019-th-non-dependent-hypothesis-in-current-goal-even-after-head-reduction","No \u2018natural\u2019-th non dependent hypothesis in current goal even after head-reduction"],[46,0,1,"coq:exn.Non-exhaustive-pattern-matching","Non exhaustive pattern matching"],[9,0,1,"coq:exn.Non-extensible-universe-declaration-not-supported-with-monomorphic-Program-Definition","Non extensible universe declaration not supported with monomorphic Program Definition"],[34,0,1,"coq:exn.Non-strictly-positive-occurrence-of-\u2018ident\u2019-in-\u2018type\u2019","Non strictly positive occurrence of \u2018ident\u2019 in \u2018type\u2019"],[14,7,1,"coq:attr.NonCumulative","NonCumulative"],[67,4,1,"coq:flag.Nonrecursive-Elimination-Schemes","Nonrecursive Elimination Schemes"],[54,0,1,"coq:exn.Not-a-context-variable","Not a context variable"],[67,0,1,"coq:exn.Not-a-discriminable-equality","Not a discriminable equality"],[67,0,1,"coq:exn.Not-a-negated-primitive-equality","Not a negated primitive equality"],[11,0,1,"coq:exn.Not-a-valid-ring-equation","Not a valid ring equation"],[54,0,1,"coq:exn.Not-a-variable-or-hypothesis","Not a variable or hypothesis"],[54,0,1,"coq:exn.Not-an-evar","Not an evar"],[58,0,1,"coq:exn.Not-an-exact-proof","Not an exact proof"],[67,0,1,"coq:exn.Not-an-inductive-goal-with-1-constructor","Not an inductive goal with 1 constructor"],[67,0,1,"coq:exn.Not-an-inductive-goal-with-2-constructors","Not an inductive goal with 2 constructors"],[67,0,1,"coq:exn.Not-an-inductive-product","Not an inductive product"],[64,0,1,"coq:exn.Not-convertible","Not convertible"],[67,0,1,"coq:exn.Not-enough-constructors","Not enough constructors"],[44,0,1,"coq:exn.Not-enough-non-implicit-arguments-to-accept-the-argument-bound-to-\u2018ident\u2019","Not enough non implicit arguments to accept the argument bound to \u2018ident\u2019"],[44,0,1,"coq:exn.Not-enough-non-implicit-arguments-to-accept-the-argument-bound-to-\u2018natural\u2019","Not enough non implicit arguments to accept the argument bound to \u2018natural\u2019"],[54,0,1,"coq:exn.Not-equal","Not equal"],[54,0,1,"coq:exn.Not-equal-(due-to-universes)","Not equal (due to universes)"],[54,0,1,"coq:exn.Not-ground","Not ground"],[72,0,1,"coq:exn.Not-the-right-number-of-induction-arguments","Not the right number of induction arguments"],[58,0,1,"coq:exn.Not-the-right-number-of-missing-arguments-(expected-\u2018natural\u2019)","Not the right number of missing arguments (expected \u2018natural\u2019)"],[71,3,1,"coq:cmd.Notation","Notation"],[71,3,1,"coq:cmd.Notation-(abbreviation)","Notation (abbreviation)"],[55,0,1,"coq:exn.Notation-levels-must-range-between-0-and-6","Notation levels must range between 0 and 6"],[67,0,1,"coq:exn.Nothing-to-inject","Nothing to inject"],[3,0,1,"coq:exn.Nothing-to-rewrite","Nothing to rewrite"],[5,4,1,"coq:flag.Nra-Cache","Nra Cache"],[71,3,1,"coq:cmd.Number-Notation","Number Notation"],[9,3,1,"coq:cmd.Obligation","Obligation"],[9,3,1,"coq:cmd.Obligation-Tactic","Obligation Tactic"],[9,3,1,"coq:cmd.Obligations","Obligations"],[64,3,1,"coq:cmd.Opaque","Opaque"],[71,3,1,"coq:cmd.Open-Scope","Open Scope"],[66,3,1,"coq:cmd.Optimize-Heap","Optimize Heap"],[66,3,1,"coq:cmd.Optimize-Proof","Optimize Proof"],[28,3,1,"coq:cmd.Parameter","Parameter"],[28,3,1,"coq:cmd.Parameters","Parameters"],[44,4,1,"coq:flag.Parsing-Explicit","Parsing Explicit"],[14,7,1,"coq:attr.Polymorphic","Polymorphic"],[14,4,1,"coq:flag.Polymorphic-Inductive-Cumulativity","Polymorphic Inductive Cumulativity"],[14,0,1,"coq:exn.Polymorphic-universe-constraints-can-only-be-declared-inside-sections,-use-Monomorphic-Constraint-instead","Polymorphic universe constraints can only be declared inside sections, use Monomorphic Constraint instead"],[14,0,1,"coq:exn.Polymorphic-universes-can-only-be-declared-inside-sections,-use-Monomorphic-Universe-instead","Polymorphic universes can only be declared inside sections, use Monomorphic Universe instead"],[59,4,1,"coq:flag.Positivity-Checking","Positivity Checking"],[57,3,1,"coq:cmd.Prenex-Implicits","Prenex Implicits"],[9,3,1,"coq:cmd.Preterm","Preterm"],[59,3,1,"coq:cmd.Primitive","Primitive"],[37,4,1,"coq:flag.Primitive-Projections","Primitive Projections"],[59,3,1,"coq:cmd.Print","Print"],[59,3,1,"coq:cmd.Print-All","Print All"],[59,3,1,"coq:cmd.Print-All-Dependencies","Print All Dependencies"],[59,3,1,"coq:cmd.Print-Assumptions","Print Assumptions"],[42,3,1,"coq:cmd.Print-Canonical-Projections","Print Canonical Projections"],[4,3,1,"coq:cmd.Print-Classes","Print Classes"],[4,3,1,"coq:cmd.Print-Coercion-Paths","Print Coercion Paths"],[4,3,1,"coq:cmd.Print-Coercions","Print Coercions"],[71,3,1,"coq:cmd.Print-Custom-Grammar","Print Custom Grammar"],[66,3,1,"coq:cmd.Print-Debug-GC","Print Debug GC"],[64,3,1,"coq:cmd.Print-Equivalent-Keys","Print Equivalent Keys"],[2,3,1,"coq:cmd.Print-Extraction-Blacklist","Print Extraction Blacklist"],[2,3,1,"coq:cmd.Print-Extraction-Callback","Print Extraction Callback"],[2,3,1,"coq:cmd.Print-Extraction-Foreign","Print Extraction Foreign"],[2,3,1,"coq:cmd.Print-Extraction-Inline","Print Extraction Inline"],[11,3,1,"coq:cmd.Print-Fields","Print Fields"],[62,3,1,"coq:cmd.Print-Firstorder-Solver","Print Firstorder Solver"],[71,3,1,"coq:cmd.Print-Grammar","Print Grammar"],[4,3,1,"coq:cmd.Print-Graph","Print Graph"],[60,3,1,"coq:cmd.Print-Hint","Print Hint"],[60,3,1,"coq:cmd.Print-HintDb","Print HintDb"],[44,3,1,"coq:cmd.Print-Implicit","Print Implicit"],[13,3,1,"coq:cmd.Print-Instances","Print Instances"],[71,3,1,"coq:cmd.Print-Keywords","Print Keywords"],[59,3,1,"coq:cmd.Print-Libraries","Print Libraries"],[59,3,1,"coq:cmd.Print-LoadPath","Print LoadPath"],[54,3,1,"coq:cmd.Print-Ltac","Print Ltac"],[54,3,1,"coq:cmd.Print-Ltac-Signatures","Print Ltac Signatures"],[55,3,1,"coq:cmd.Print-Ltac2","Print Ltac2"],[55,3,1,"coq:cmd.Print-Ltac2-Signatures","Print Ltac2 Signatures"],[55,3,1,"coq:cmd.Print-Ltac2-Type","Print Ltac2 Type"],[59,3,1,"coq:cmd.Print-ML-Modules","Print ML Modules"],[59,3,1,"coq:cmd.Print-ML-Path","Print ML Path"],[35,3,1,"coq:cmd.Print-Module","Print Module"],[35,3,1,"coq:cmd.Print-Module-Type","Print Module Type"],[35,3,1,"coq:cmd.Print-Namespace","Print Namespace"],[71,3,1,"coq:cmd.Print-Notation","Print Notation"],[59,3,1,"coq:cmd.Print-Opaque-Dependencies","Print Opaque Dependencies"],[29,3,1,"coq:cmd.Print-Options","Print Options"],[59,3,1,"coq:cmd.Print-Registered","Print Registered"],[59,3,1,"coq:cmd.Print-Registered-Schemes","Print Registered Schemes"],[60,3,1,"coq:cmd.Print-Rewrite-HintDb","Print Rewrite HintDb"],[11,3,1,"coq:cmd.Print-Rings","Print Rings"],[71,3,1,"coq:cmd.Print-Scope","Print Scope"],[71,3,1,"coq:cmd.Print-Scopes","Print Scopes"],[59,3,1,"coq:cmd.Print-Section","Print Section"],[64,3,1,"coq:cmd.Print-Strategies","Print Strategies"],[64,3,1,"coq:cmd.Print-Strategy","Print Strategy"],[29,3,1,"coq:cmd.Print-Table","Print Table"],[29,3,1,"coq:cmd.Print-Tables","Print Tables"],[59,3,1,"coq:cmd.Print-Transparent-Dependencies","Print Transparent Dependencies"],[13,3,1,"coq:cmd.Print-Typeclasses","Print Typeclasses"],[59,3,1,"coq:cmd.Print-Typing-Flags","Print Typing Flags"],[14,3,1,"coq:cmd.Print-Universes","Print Universes"],[71,3,1,"coq:cmd.Print-Visibility","Print Visibility"],[59,4,1,"coq:flag.Printing-All","Printing All"],[46,4,1,"coq:flag.Printing-Allow-Match-Default-Clause","Printing Allow Match Default Clause"],[4,8,1,"coq:table.Printing-Coercion","Printing Coercion"],[4,4,1,"coq:flag.Printing-Coercions","Printing Coercions"],[59,4,1,"coq:flag.Printing-Compact-Contexts","Printing Compact Contexts"],[37,8,1,"coq:table.Printing-Constructor","Printing Constructor"],[59,4,1,"coq:flag.Printing-Dependent-Evars-Line","Printing Dependent Evars Line"],[59,6,1,"coq:opt.Printing-Depth","Printing Depth"],[43,4,1,"coq:flag.Printing-Existential-Instances","Printing Existential Instances"],[46,4,1,"coq:flag.Printing-Factorizable-Match-Patterns","Printing Factorizable Match Patterns"],[27,4,1,"coq:flag.Printing-Float","Printing Float"],[66,4,1,"coq:flag.Printing-Goal-Names","Printing Goal Names"],[66,4,1,"coq:flag.Printing-Goal-Tags","Printing Goal Tags"],[46,8,1,"coq:table.Printing-If","Printing If"],[44,4,1,"coq:flag.Printing-Implicit","Printing Implicit"],[44,4,1,"coq:flag.Printing-Implicit-Defensive","Printing Implicit Defensive"],[46,8,1,"coq:table.Printing-Let","Printing Let"],[46,4,1,"coq:flag.Printing-Match-All-Subterms","Printing Match All Subterms"],[46,4,1,"coq:flag.Printing-Matching","Printing Matching"],[71,4,1,"coq:flag.Printing-Notations","Printing Notations"],[71,4,1,"coq:flag.Printing-Parentheses","Printing Parentheses"],[37,4,1,"coq:flag.Printing-Primitive-Projection-Parameters","Printing Primitive Projection Parameters"],[37,4,1,"coq:flag.Printing-Projections","Printing Projections"],[71,4,1,"coq:flag.Printing-Raw-Literals","Printing Raw Literals"],[37,8,1,"coq:table.Printing-Record","Printing Record"],[37,4,1,"coq:flag.Printing-Records","Printing Records"],[12,4,1,"coq:flag.Printing-Relevance-Marks","Printing Relevance Marks"],[46,4,1,"coq:flag.Printing-Synth","Printing Synth"],[59,4,1,"coq:flag.Printing-Unfocused","Printing Unfocused"],[37,4,1,"coq:flag.Printing-Unfolded-Projection-As-Match","Printing Unfolded Projection As Match"],[14,4,1,"coq:flag.Printing-Universes","Printing Universes"],[44,4,1,"coq:flag.Printing-Use-Implicit-Types","Printing Use Implicit Types"],[59,6,1,"coq:opt.Printing-Width","Printing Width"],[46,4,1,"coq:flag.Printing-Wildcard","Printing Wildcard"],[40,7,1,"coq:attr.Private","Private"],[14,4,1,"coq:flag.Private-Polymorphic-Universes","Private Polymorphic Universes"],[59,3,1,"coq:cmd.Profile","Profile"],[9,7,1,"coq:attr.Program","Program"],[9,4,1,"coq:flag.Program-Cases","Program Cases"],[9,4,1,"coq:flag.Program-Generalized-Coercion","Program Generalized Coercion"],[9,4,1,"coq:flag.Program-Mode","Program Mode"],[66,3,1,"coq:cmd.Proof","Proof"],[66,3,1,"coq:cmd.Proof-Mode","Proof Mode"],[66,3,1,"coq:cmd.Proof-`term`","Proof `term`"],[66,3,1,"coq:cmd.Proof-using","Proof using"],[60,3,1,"coq:cmd.Proof-with","Proof with"],[32,3,1,"coq:cmd.Property","Property"],[32,3,1,"coq:cmd.Proposition","Proposition"],[5,5,1,"coq:thm.Psatz","Psatz"],[2,3,1,"coq:cmd.Pwd","Pwd"],[66,3,1,"coq:cmd.Qed","Qed"],[59,3,1,"coq:cmd.Quit","Quit"],[37,3,1,"coq:cmd.Record","Record"],[37,0,1,"coq:exn.Records-declared-with-the-keyword-Record-or-Structure-cannot-be-recursive","Records declared with the keyword Record or Structure cannot be recursive"],[2,3,1,"coq:cmd.Recursive-Extraction","Recursive Extraction"],[2,3,1,"coq:cmd.Recursive-Extraction-Library","Recursive Extraction Library"],[59,3,1,"coq:cmd.Redirect","Redirect"],[59,3,1,"coq:cmd.Register","Register"],[59,3,1,"coq:cmd.Register-Inline","Register Inline"],[59,3,1,"coq:cmd.Register-Scheme","Register Scheme"],[64,4,1,"coq:flag.Regular-Subst-Tactic","Regular Subst Tactic"],[32,3,1,"coq:cmd.Remark","Remark"],[29,3,1,"coq:cmd.Remove","Remove"],[60,3,1,"coq:cmd.Remove-Hints","Remove Hints"],[59,3,1,"coq:cmd.Require","Require"],[59,3,1,"coq:cmd.Require-Export","Require Export"],[59,3,1,"coq:cmd.Require-Import","Require Import"],[71,3,1,"coq:cmd.Reserved-Infix","Reserved Infix"],[71,3,1,"coq:cmd.Reserved-Notation","Reserved Notation"],[59,3,1,"coq:cmd.Reset","Reset"],[2,3,1,"coq:cmd.Reset-Extraction-Blacklist","Reset Extraction Blacklist"],[2,3,1,"coq:cmd.Reset-Extraction-Callback","Reset Extraction Callback"],[2,3,1,"coq:cmd.Reset-Extraction-Inline","Reset Extraction Inline"],[59,3,1,"coq:cmd.Reset-Initial","Reset Initial"],[54,3,1,"coq:cmd.Reset-Ltac-Profile","Reset Ltac Profile"],[66,3,1,"coq:cmd.Restart","Restart"],[44,4,1,"coq:flag.Reversible-Pattern-Implicit","Reversible Pattern Implicit"],[10,3,1,"coq:cmd.Rewrite-Rule","Rewrite Rule"],[10,3,1,"coq:cmd.Rewrite-Rules","Rewrite Rules"],[10,0,1,"coq:exn.Rewrite-rule-declaration-requires-passing-the-flag-\"-allow-rewrite-rules\"","Rewrite rule declaration requires passing the flag "-allow-rewrite-rules""],[67,4,1,"coq:flag.Rewriting-Schemes","Rewriting Schemes"],[11,0,1,"coq:exn.Ring-operation-should-be-declared-as-a-morphism","Ring operation should be declared as a morphism"],[12,0,1,"coq:exn.SProp-is-disallowed-because-the-\"Allow-StrictProp\"-flag-is-off","SProp is disallowed because the "Allow StrictProp" flag is off"],[66,3,1,"coq:cmd.Save","Save"],[67,3,1,"coq:cmd.Scheme","Scheme"],[67,3,1,"coq:cmd.Scheme-Boolean-Equality","Scheme Boolean Equality"],[67,3,1,"coq:cmd.Scheme-Equality","Scheme Equality"],[71,0,1,"coq:exn.Scope-delimiters-should-not-start-with-an-underscore","Scope delimiters should not start with an underscore"],[71,0,1,"coq:exn.Scope-names-should-not-start-with-an-underscore","Scope names should not start with an underscore"],[59,3,1,"coq:cmd.Search","Search"],[59,8,1,"coq:table.Search-Blacklist","Search Blacklist"],[59,4,1,"coq:flag.Search-Output-Name-Only","Search Output Name Only"],[59,3,1,"coq:cmd.SearchPattern","SearchPattern"],[59,3,1,"coq:cmd.SearchRewrite","SearchRewrite"],[38,3,1,"coq:cmd.Section","Section"],[64,0,1,"coq:exn.Section-variable-\u2018ident\u2019-occurs-implicitly-in-global-declaration-\u2018qualid\u2019-present-in-hypothesis-\u2018ident\u2019","Section variable \u2018ident\u2019 occurs implicitly in global declaration \u2018qualid\u2019 present in hypothesis \u2018ident\u2019"],[64,0,1,"coq:exn.Section-variable-\u2018ident\u2019-occurs-implicitly-in-global-declaration-\u2018qualid\u2019-present-in-the-conclusion","Section variable \u2018ident\u2019 occurs implicitly in global declaration \u2018qualid\u2019 present in the conclusion"],[2,3,1,"coq:cmd.Separate-Extraction","Separate Extraction"],[29,3,1,"coq:cmd.Set","Set"],[35,4,1,"coq:flag.Short-Module-Printing","Short Module Printing"],[66,3,1,"coq:cmd.Show","Show"],[66,3,1,"coq:cmd.Show-Conjectures","Show Conjectures"],[66,3,1,"coq:cmd.Show-Existentials","Show Existentials"],[2,3,1,"coq:cmd.Show-Extraction","Show Extraction"],[66,3,1,"coq:cmd.Show-Goal","Show Goal"],[66,3,1,"coq:cmd.Show-Intro","Show Intro"],[66,3,1,"coq:cmd.Show-Intros","Show Intros"],[5,3,1,"coq:cmd.Show-Lia-Profile","Show Lia Profile"],[54,3,1,"coq:cmd.Show-Ltac-Profile","Show Ltac Profile"],[66,3,1,"coq:cmd.Show-Match","Show Match"],[9,3,1,"coq:cmd.Show-Obligation-Tactic","Show Obligation Tactic"],[66,3,1,"coq:cmd.Show-Proof","Show Proof"],[66,3,1,"coq:cmd.Show-Universes","Show Universes"],[5,3,1,"coq:cmd.Show-Zify","Show Zify"],[35,0,1,"coq:exn.Signature-components-for-field-\u2018ident\u2019-do-not-match","Signature components for field \u2018ident\u2019 do not match"],[59,4,1,"coq:flag.Silent","Silent"],[9,3,1,"coq:cmd.Solve-All-Obligations","Solve All Obligations"],[9,3,1,"coq:cmd.Solve-Obligations","Solve Obligations"],[66,4,1,"coq:flag.Solve-Unification-Constraints","Solve Unification Constraints"],[57,4,1,"coq:flag.SsrHave-NoTCResolution","SsrHave NoTCResolution"],[57,4,1,"coq:flag.SsrIdents","SsrIdents"],[57,4,1,"coq:flag.SsrOldRewriteGoalsOrder","SsrOldRewriteGoalsOrder"],[57,4,1,"coq:flag.SsrRewrite","SsrRewrite"],[71,2,1,"coq:warn.Stack-overflow-or-segmentation-fault-happens-when-working-with-large-numbers-in-\u2018type\u2019-(threshold-may-vary-depending-on-your-system-limits-and-on-the-command-executed)","Stack overflow or segmentation fault happens when working with large numbers in \u2018type\u2019 (threshold may vary depending on your system limits and on the command executed)"],[64,3,1,"coq:cmd.Strategy","Strategy"],[44,4,1,"coq:flag.Strict-Implicit","Strict Implicit"],[14,4,1,"coq:flag.Strict-Universe-Declaration","Strict Universe Declaration"],[71,3,1,"coq:cmd.String-Notation","String Notation"],[44,4,1,"coq:flag.Strongly-Strict-Implicit","Strongly Strict Implicit"],[67,4,1,"coq:flag.Structural-Injection","Structural Injection"],[37,3,1,"coq:cmd.Structure","Structure"],[4,3,1,"coq:cmd.SubClass","SubClass"],[59,3,1,"coq:cmd.Succeed","Succeed"],[66,4,1,"coq:flag.Suggest-Proof-Using","Suggest Proof Using"],[10,3,1,"coq:cmd.Symbol","Symbol"],[10,3,1,"coq:cmd.Symbols","Symbols"],[71,0,1,"coq:exn.Syntax-error:-[prim:reference]-expected-after-'Notation'-(in-[vernac:command])","Syntax error: [prim:reference] expected after 'Notation' (in [vernac:command])"],[71,0,1,"coq:exn.Syntax-error:-[prim:reference]-expected-after-[prim:reference]-(in-[vernac:command])","Syntax error: [prim:reference] expected after [prim:reference] (in [vernac:command])"],[71,3,1,"coq:cmd.Tactic-Notation","Tactic Notation"],[54,0,1,"coq:exn.Tactic-failure","Tactic failure"],[54,0,1,"coq:exn.Tactic-failure-(level-\u2018natural\u2019)","Tactic failure (level \u2018natural\u2019)"],[54,0,1,"coq:exn.Tactic-failure:--succeeds","Tactic failure: <tactic closure> succeeds"],[64,0,1,"coq:exn.Tactic-failure:-Setoid-library-not-loaded","Tactic failure: Setoid library not loaded"],[64,0,1,"coq:exn.Tactic-generated-a-subgoal-identical-to-the-original-goal","Tactic generated a subgoal identical to the original goal"],[64,0,1,"coq:exn.Terms-do-not-have-convertible-types","Terms do not have convertible types"],[29,3,1,"coq:cmd.Test","Test"],[60,0,1,"coq:exn.The-\"at\"-syntax-isn't-available-yet-for-the-autorewrite-tactic","The "at" syntax isn't available yet for the autorewrite tactic"],[41,0,1,"coq:exn.The-&-modifier-may-only-occur-once","The & modifier may only occur once"],[71,2,1,"coq:warn.The-'abstract-after'-directive-has-no-effect-when-the-parsing-function-(\u2018qualid\u2019)-targets-an-option-type","The 'abstract after' directive has no effect when the parsing function (\u2018qualid\u2019) targets an option type"],[41,0,1,"coq:exn.The-'clear-implicits'-flag-must-be-omitted-if-implicit-annotations-are-given","The 'clear implicits' flag must be omitted if implicit annotations are given"],[41,0,1,"coq:exn.The-'default-implicits'-flag-is-incompatible-with-implicit-annotations","The 'default implicits' flag is incompatible with implicit annotations"],[41,0,1,"coq:exn.The-/-modifier-may-only-occur-once","The / modifier may only occur once"],[59,0,1,"coq:exn.The-command-has-not-failed!","The command has not failed!"],[34,0,1,"coq:exn.The-conclusion-of-\u2018type\u2019-is-not-valid;-it-must-be-built-from-\u2018ident\u2019","The conclusion of \u2018type\u2019 is not valid; it must be built from \u2018ident\u2019"],[46,0,1,"coq:exn.The-constructor-\u2018ident\u2019-expects-\u2018natural\u2019-arguments","The constructor \u2018ident\u2019 expects \u2018natural\u2019 arguments"],[14,0,1,"coq:exn.The-cumulative-attribute-can-only-be-used-in-a-polymorphic-context","The cumulative attribute can only be used in a polymorphic context"],[46,0,1,"coq:exn.The-elimination-predicate-term-should-be-of-arity-\u2018natural\u2019-(for-non-dependent-case)-or-\u2018natural\u2019-(for-dependent-case)","The elimination predicate term should be of arity \u2018natural\u2019 (for non dependent case) or \u2018natural\u2019 (for dependent case)"],[35,0,1,"coq:exn.The-field-\u2018ident\u2019-is-missing-in-\u2018qualid\u2019","The field \u2018ident\u2019 is missing in \u2018qualid\u2019"],[72,0,1,"coq:exn.The-recursive-argument-must-be-specified","The recursive argument must be specified"],[55,0,1,"coq:exn.The-reference-X-was-not-found-in-the-current-environment","The reference X was not found in the current environment"],[64,0,1,"coq:exn.The-reference-is-not-unfoldable","The reference is not unfoldable"],[64,0,1,"coq:exn.The-reference-\u2018qualid\u2019-was-not-found-in-the-current-environment","The reference \u2018qualid\u2019 was not found in the current environment"],[58,0,1,"coq:exn.The-term-\"\u2018type\u2019\"-has-type-\"\u2018type\u2019\"-which-should-be-Set,-Prop-or-Type","The term "\u2018type\u2019" has type "\u2018type\u2019" which should be Set, Prop or Type"],[2,0,1,"coq:exn.The-term-\u2018qualid\u2019-is-already-defined-as-foreign-custom-constant","The term \u2018qualid\u2019 is already defined as foreign custom constant"],[2,0,1,"coq:exn.The-term-\u2018qualid\u2019-is-already-defined-as-inline-custom-constant","The term \u2018qualid\u2019 is already defined as inline custom constant"],[32,0,1,"coq:exn.The-term-\u2018term\u2019-has-type-\u2018type\u2019-which-should-be-Set,-Prop-or-Type","The term \u2018term\u2019 has type \u2018type\u2019 which should be Set, Prop or Type"],[32,0,1,"coq:exn.The-term-\u2018term\u2019-has-type-\u2018type\u2019-while-it-is-expected-to-have-type-\u2018type\u2019'","The term \u2018term\u2019 has type \u2018type\u2019 while it is expected to have type \u2018type\u2019'"],[67,0,1,"coq:exn.The-type-has-no-constructors","The type has no constructors"],[59,0,1,"coq:exn.The-type-\u2018ident\u2019-must-be-registered-before-this-construction-can-be-typechecked","The type \u2018ident\u2019 must be registered before this construction can be typechecked"],[46,0,1,"coq:exn.The-variable-ident-is-bound-several-times-in-pattern-term","The variable ident is bound several times in pattern term"],[58,0,1,"coq:exn.The-variable-\u2018ident\u2019-is-already-declared","The variable \u2018ident\u2019 is already declared"],[40,0,1,"coq:exn.The-\u2018natural\u2019-th-argument-of-\u2018ident\u2019-must-be-\u2018ident\u2019-in-\u2018type\u2019","The \u2018natural\u2019 th argument of \u2018ident\u2019 must be \u2018ident\u2019 in \u2018type\u2019"],[32,3,1,"coq:cmd.Theorem","Theorem"],[54,0,1,"coq:exn.There-is-already-an-Ltac-named-\u2018qualid\u2019","There is already an Ltac named \u2018qualid\u2019"],[54,0,1,"coq:exn.There-is-no-Ltac-named-\u2018qualid\u2019","There is no Ltac named \u2018qualid\u2019"],[29,2,1,"coq:warn.There-is-no-flag-or-option-with-this-name:-\"\u2018setting_name\u2019\"","There is no flag or option with this name: "\u2018setting_name\u2019""],[29,0,1,"coq:exn.There-is-no-flag,-option-or-table-with-this-name:-\"\u2018setting_name\u2019\"","There is no flag, option or table with this name: "\u2018setting_name\u2019""],[29,0,1,"coq:exn.There-is-no-qualid-valued-table-with-this-name:-\"\u2018setting_name\u2019\"","There is no qualid-valued table with this name: "\u2018setting_name\u2019""],[29,0,1,"coq:exn.There-is-no-string-valued-table-with-this-name:-\"\u2018setting_name\u2019\"","There is no string-valued table with this name: "\u2018setting_name\u2019""],[38,0,1,"coq:exn.There-is-nothing-to-end","There is nothing to end"],[29,2,1,"coq:warn.This-command-does-not-support-this-attribute","This command does not support this attribute"],[59,0,1,"coq:exn.This-object-does-not-support-universe-names","This object does not support universe names"],[66,0,1,"coq:exn.This-proof-is-focused,-but-cannot-be-unfocused-this-way","This proof is focused, but cannot be unfocused this way"],[54,0,1,"coq:exn.This-tactic-has-more-than-one-success","This tactic has more than one success"],[59,3,1,"coq:cmd.Time","Time"],[59,3,1,"coq:cmd.Timeout","Timeout"],[71,2,1,"coq:warn.To-avoid-stack-overflow,-large-numbers-in-\u2018type\u2019-are-interpreted-as-applications-of-\u2018qualid\u2019","To avoid stack overflow, large numbers in \u2018type\u2019 are interpreted as applications of \u2018qualid\u2019"],[41,0,1,"coq:exn.To-rename-arguments-the-'rename'-flag-must-be-specified","To rename arguments the 'rename' flag must be specified"],[64,3,1,"coq:cmd.Transparent","Transparent"],[9,4,1,"coq:flag.Transparent-Obligations","Transparent Obligations"],[35,2,1,"coq:warn.Trying-to-mask-the-absolute-name-\u2018qualid\u2019!","Trying to mask the absolute name \u2018qualid\u2019!"],[59,3,1,"coq:cmd.Type","Type"],[67,0,1,"coq:exn.Type-of-\u2018ident\u2019-is-not-an-equality-of-recognized-\u03a3-types:-expected-one-of-sig-sig2-sigT-sigT2-sigT2-ex-or-ex2-but-got-\u2018term\u2019","Type of \u2018ident\u2019 is not an equality of recognized \u03a3 types: expected one of sig sig2 sigT sigT2 sigT2 ex or ex2 but got \u2018term\u2019"],[13,4,1,"coq:flag.Typeclass-Resolution-For-Conversion","Typeclass Resolution For Conversion"],[13,4,1,"coq:flag.Typeclasses-Debug","Typeclasses Debug"],[13,6,1,"coq:opt.Typeclasses-Debug-Verbosity","Typeclasses Debug Verbosity"],[13,6,1,"coq:opt.Typeclasses-Default-Mode","Typeclasses Default Mode"],[13,4,1,"coq:flag.Typeclasses-Dependency-Order","Typeclasses Dependency Order"],[13,6,1,"coq:opt.Typeclasses-Depth","Typeclasses Depth"],[13,4,1,"coq:flag.Typeclasses-Iterative-Deepening","Typeclasses Iterative Deepening"],[13,4,1,"coq:flag.Typeclasses-Limit-Intros","Typeclasses Limit Intros"],[13,3,1,"coq:cmd.Typeclasses-Opaque","Typeclasses Opaque"],[13,4,1,"coq:flag.Typeclasses-Strict-Resolution","Typeclasses Strict Resolution"],[13,3,1,"coq:cmd.Typeclasses-Transparent","Typeclasses Transparent"],[13,4,1,"coq:flag.Typeclasses-Unique-Instances","Typeclasses Unique Instances"],[13,4,1,"coq:flag.Typeclasses-Unique-Solutions","Typeclasses Unique Solutions"],[13,3,1,"coq:cmd.Typeclasses-eauto","Typeclasses eauto"],[67,0,1,"coq:exn.Unable-to-find-an-instance-for-the-variables-\u2018ident\u2019-\u2026-\u2018ident\u2019","Unable to find an instance for the variables \u2018ident\u2019 \u2026 \u2018ident\u2019"],[58,0,1,"coq:exn.Unable-to-find-an-instance-for-the-variables-\u2018ident\u2019\u2026\u2018ident\u2019","Unable to find an instance for the variables \u2018ident\u2019\u2026\u2018ident\u2019"],[46,0,1,"coq:exn.Unable-to-infer-a-match-predicate","Unable to infer a match predicate"],[3,0,1,"coq:exn.Unable-to-satisfy-the-rewriting-constraints","Unable to satisfy the rewriting constraints"],[58,0,1,"coq:exn.Unable-to-unify-\u2018one_term\u2019-with-\u2018one_term\u2019","Unable to unify \u2018one_term\u2019 with \u2018one_term\u2019"],[55,0,1,"coq:exn.Unbound-[value|constructor]-X","Unbound [value|constructor] X"],[54,0,1,"coq:exn.Unbound-context-identifier-\u2018ident\u2019","Unbound context identifier \u2018ident\u2019"],[14,0,1,"coq:exn.Undeclared-universe-\u2018ident\u2019","Undeclared universe \u2018ident\u2019"],[71,3,1,"coq:cmd.Undelimit-Scope","Undelimit Scope"],[66,3,1,"coq:cmd.Undo","Undo"],[71,0,1,"coq:exn.Unexpected-non-option-term-\u2018term\u2019-while-parsing-a-number-notation","Unexpected non-option term \u2018term\u2019 while parsing a number notation"],[71,0,1,"coq:exn.Unexpected-non-option-term-\u2018term\u2019-while-parsing-a-string-notation","Unexpected non-option term \u2018term\u2019 while parsing a string notation"],[71,0,1,"coq:exn.Unexpected-only-parsing-for-an-only-printing-notation","Unexpected only parsing for an only printing notation"],[71,0,1,"coq:exn.Unexpected-only-printing-for-an-only-parsing-notation","Unexpected only printing for an only parsing notation"],[71,0,1,"coq:exn.Unexpected-term-\u2018term\u2019-while-parsing-a-number-notation","Unexpected term \u2018term\u2019 while parsing a number notation"],[71,0,1,"coq:exn.Unexpected-term-\u2018term\u2019-while-parsing-a-string-notation","Unexpected term \u2018term\u2019 while parsing a string notation"],[66,3,1,"coq:cmd.Unfocus","Unfocus"],[66,3,1,"coq:cmd.Unfocused","Unfocused"],[34,4,1,"coq:flag.Uniform-Inductive-Parameters","Uniform Inductive Parameters"],[14,3,1,"coq:cmd.Universe","Universe"],[59,4,1,"coq:flag.Universe-Checking","Universe Checking"],[14,4,1,"coq:flag.Universe-Minimization-ToSet","Universe Minimization ToSet"],[14,4,1,"coq:flag.Universe-Polymorphism","Universe Polymorphism"],[14,0,1,"coq:exn.Universe-inconsistency","Universe inconsistency"],[59,0,1,"coq:exn.Universe-instance-length-is-\u2018natural\u2019-but-should-be-\u2018natural\u2019","Universe instance length is \u2018natural\u2019 but should be \u2018natural\u2019"],[14,3,1,"coq:cmd.Universes","Universes"],[71,0,1,"coq:exn.Unknown-custom-entry","Unknown custom entry"],[71,0,1,"coq:exn.Unknown-custom-entry:-\u2018ident\u2019","Unknown custom entry: \u2018ident\u2019"],[66,0,1,"coq:exn.Unknown-inductive-type","Unknown inductive type"],[29,3,1,"coq:cmd.Unset","Unset"],[66,3,1,"coq:cmd.Unshelve","Unshelve"],[71,0,1,"coq:exn.Unterminated-string-in-notation","Unterminated string in notation"],[28,2,1,"coq:warn.Use-of-\"Variable\"-or-\"Hypothesis\"-outside-sections-behaves-as-\"#[local]-Parameter\"-or-\"#[local]-Axiom\"","Use of "Variable" or "Hypothesis" outside sections behaves as "#[local] Parameter" or "#[local] Axiom""],[71,2,1,"coq:warn.Use-of-\u2018string\u2019-Notation-is-deprecated-as-it-is-inconsistent-with-pattern-syntax","Use of \u2018string\u2019 Notation is deprecated as it is inconsistent with pattern syntax"],[13,2,1,"coq:warn.Using-inferred-default-mode:-\u201cmode\u201d-for-\u201c\u2018ident\u2019\u201d","Using inferred default mode: \u201cmode\u201d for \u201c\u2018ident\u2019\u201d"],[66,3,1,"coq:cmd.Validate-Proof","Validate Proof"],[28,3,1,"coq:cmd.Variable","Variable"],[66,2,1,"coq:warn.Variable-All-is-shadowed-by-Collection-named-All-containing-all-variables","Variable All is shadowed by Collection named All containing all variables"],[28,3,1,"coq:cmd.Variables","Variables"],[40,3,1,"coq:cmd.Variant","Variant"],[59,6,1,"coq:opt.Warnings","Warnings"],[44,0,1,"coq:exn.Wrong-argument-name","Wrong argument name"],[44,0,1,"coq:exn.Wrong-argument-position","Wrong argument position"],[66,0,1,"coq:exn.Wrong-bullet-\u2018bullet\u2019:-Bullet-\u2018bullet\u2019-is-mandatory-here","Wrong bullet \u2018bullet\u2019: Bullet \u2018bullet\u2019 is mandatory here"],[66,0,1,"coq:exn.Wrong-bullet-\u2018bullet\u2019:-Current-bullet-\u2018bullet\u2019-is-not-finished","Wrong bullet \u2018bullet\u2019: Current bullet \u2018bullet\u2019 is not finished"],[54,1,1,"coq:tacn.[-\u2026-|-\u2026-|-\u2026-]-(dispatch)","[ \u2026 | \u2026 | \u2026 ] (dispatch)"],[54,1,1,"coq:tacn.[>-\u2026-|-\u2026-|-\u2026-]-(dispatch)","[> \u2026 | \u2026 | \u2026 ] (dispatch)"],[55,7,1,"coq:attr.abstract","abstract"],[66,1,1,"coq:tacn.abstract","abstract"],[57,1,1,"coq:tacn.abstract-(ssreflect)","abstract (ssreflect)"],[58,1,1,"coq:tacn.absurd","absurd"],[71,7,1,"coq:attr.add_bottom","add_bottom"],[71,7,1,"coq:attr.add_top","add_top"],[66,1,1,"coq:tacn.admit","admit"],[58,1,1,"coq:tacn.apply","apply"],[57,1,1,"coq:tacn.apply-(ssreflect)","apply (ssreflect)"],[58,1,1,"coq:tacn.assert","assert"],[54,1,1,"coq:tacn.assert_fails","assert_fails"],[54,1,1,"coq:tacn.assert_succeeds","assert_succeeds"],[58,1,1,"coq:tacn.assumption","assumption"],[60,1,1,"coq:tacn.auto","auto"],[13,1,1,"coq:tacn.autoapply","autoapply"],[34,2,1,"coq:warn.automatic-prop-lowering","automatic-prop-lowering"],[60,1,1,"coq:tacn.autorewrite","autorewrite"],[60,1,1,"coq:tacn.autounfold","autounfold"],[60,1,1,"coq:tacn.autounfold_one","autounfold_one"],[62,1,1,"coq:tacn.btauto","btauto"],[66,1,1,"coq:tacn.bullet-(--+-*)","bullet (- + *)"],[57,1,1,"coq:tacn.by","by"],[59,7,1,"coq:attr.bypass_check(guard)","bypass_check(guard)"],[59,7,1,"coq:attr.bypass_check(positivity)","bypass_check(positivity)"],[59,7,1,"coq:attr.bypass_check(universes)","bypass_check(universes)"],[42,7,1,"coq:attr.canonical","canonical"],[67,1,1,"coq:tacn.case","case"],[57,1,1,"coq:tacn.case-(ssreflect)","case (ssreflect)"],[67,1,1,"coq:tacn.case_eq","case_eq"],[64,1,1,"coq:tacn.cbn","cbn"],[64,1,1,"coq:tacn.cbv","cbv"],[64,1,1,"coq:tacn.change","change"],[64,1,1,"coq:tacn.change_no_check","change_no_check"],[58,1,1,"coq:tacn.classical_left","classical_left"],[58,1,1,"coq:tacn.classical_right","classical_right"],[58,1,1,"coq:tacn.clear","clear"],[58,1,1,"coq:tacn.clear-dependent","clear dependent"],[38,7,1,"coq:attr.clearbody","clearbody"],[58,1,1,"coq:tacn.clearbody","clearbody"],[71,2,1,"coq:warn.closed-notation-not-level-0","closed-notation-not-level-0"],[67,1,1,"coq:tacn.cofix","cofix"],[67,1,1,"coq:tacn.compare","compare"],[64,1,1,"coq:tacn.compute","compute"],[57,1,1,"coq:tacn.congr","congr"],[62,1,1,"coq:tacn.congruence","congruence"],[54,1,1,"coq:tacn.constr_eq","constr_eq"],[54,1,1,"coq:tacn.constr_eq_nounivs","constr_eq_nounivs"],[54,1,1,"coq:tacn.constr_eq_strict","constr_eq_strict"],[67,1,1,"coq:tacn.constructor","constructor"],[54,1,1,"coq:tacn.context","context"],[58,1,1,"coq:tacn.contradict","contradict"],[58,1,1,"coq:tacn.contradiction","contradiction"],[54,1,1,"coq:tacn.convert","convert"],[58,1,1,"coq:tacn.cut","cut"],[66,1,1,"coq:tacn.cycle","cycle"],[60,1,1,"coq:tacn.debug-auto","debug auto"],[60,1,1,"coq:tacn.debug-eauto","debug eauto"],[60,1,1,"coq:tacn.debug-trivial","debug trivial"],[67,1,1,"coq:tacn.decide","decide"],[67,1,1,"coq:tacn.decide-equality","decide equality"],[67,1,1,"coq:tacn.decompose","decompose"],[67,1,1,"coq:tacn.decompose-record","decompose record"],[67,1,1,"coq:tacn.decompose-sum","decompose sum"],[67,1,1,"coq:tacn.dependent-destruction","dependent destruction"],[58,1,1,"coq:tacn.dependent-generalize_eqs","dependent generalize_eqs"],[58,1,1,"coq:tacn.dependent-generalize_eqs_vars","dependent generalize_eqs_vars"],[67,1,1,"coq:tacn.dependent-induction","dependent induction"],[67,1,1,"coq:tacn.dependent-inversion","dependent inversion"],[67,1,1,"coq:tacn.dependent-inversion_clear","dependent inversion_clear"],[67,1,1,"coq:tacn.dependent-rewrite","dependent rewrite"],[67,1,1,"coq:tacn.dependent-simple-inversion","dependent simple inversion"],[74,7,1,"coq:attr.deprecated","deprecated"],[67,1,1,"coq:tacn.destauto","destauto"],[67,1,1,"coq:tacn.destruct","destruct"],[60,1,1,"coq:tacn.dfs-eauto","dfs eauto"],[62,1,1,"coq:tacn.dintuition","dintuition"],[27,1,1,"coq:tacn.discrR","discrR"],[67,1,1,"coq:tacn.discriminate","discriminate"],[54,1,1,"coq:tacn.do","do"],[57,1,1,"coq:tacn.do-(ssreflect)","do (ssreflect)"],[57,1,1,"coq:tacn.done","done"],[62,1,1,"coq:tacn.dtauto","dtauto"],[58,1,1,"coq:tacn.eapply","eapply"],[58,1,1,"coq:tacn.eassert","eassert"],[58,1,1,"coq:tacn.eassumption","eassumption"],[60,1,1,"coq:tacn.easy","easy"],[60,1,1,"coq:tacn.eauto","eauto"],[67,1,1,"coq:tacn.ecase","ecase"],[67,1,1,"coq:tacn.econstructor","econstructor"],[67,1,1,"coq:tacn.edestruct","edestruct"],[67,1,1,"coq:tacn.ediscriminate","ediscriminate"],[67,1,1,"coq:tacn.eelim","eelim"],[58,1,1,"coq:tacn.eenough","eenough"],[58,1,1,"coq:tacn.eexact","eexact"],[67,1,1,"coq:tacn.eexists","eexists"],[67,1,1,"coq:tacn.einduction","einduction"],[67,1,1,"coq:tacn.einjection","einjection"],[58,1,1,"coq:tacn.eintros","eintros"],[67,1,1,"coq:tacn.eleft","eleft"],[67,1,1,"coq:tacn.elim","elim"],[57,1,1,"coq:tacn.elim-(ssreflect)","elim (ssreflect)"],[58,1,1,"coq:tacn.enough","enough"],[58,1,1,"coq:tacn.epose","epose"],[58,1,1,"coq:tacn.epose-proof","epose proof"],[58,1,1,"coq:tacn.eremember","eremember"],[64,1,1,"coq:tacn.erewrite","erewrite"],[67,1,1,"coq:tacn.eright","eright"],[58,1,1,"coq:tacn.eset","eset"],[67,1,1,"coq:tacn.esimplify_eq","esimplify_eq"],[67,1,1,"coq:tacn.esplit","esplit"],[64,1,1,"coq:tacn.etransitivity","etransitivity"],[64,1,1,"coq:tacn.eval","eval"],[58,1,1,"coq:tacn.evar","evar"],[58,1,1,"coq:tacn.exact","exact"],[57,1,1,"coq:tacn.exact-(ssreflect)","exact (ssreflect)"],[58,1,1,"coq:tacn.exact_no_check","exact_no_check"],[54,1,1,"coq:tacn.exactly_once","exactly_once"],[58,1,1,"coq:tacn.exfalso","exfalso"],[67,1,1,"coq:tacn.exists","exists"],[35,7,1,"coq:attr.export","export"],[64,1,1,"coq:tacn.f_equal","f_equal"],[54,1,1,"coq:tacn.fail","fail"],[11,1,1,"coq:tacn.field","field"],[11,1,1,"coq:tacn.field_lookup","field_lookup"],[11,1,1,"coq:tacn.field_simplify","field_simplify"],[11,1,1,"coq:tacn.field_simplify_eq","field_simplify_eq"],[54,1,1,"coq:tacn.finish_timing","finish_timing"],[54,1,1,"coq:tacn.first","first"],[57,1,1,"coq:tacn.first-(ssreflect)","first (ssreflect)"],[57,9,1,"coq:tacv.first-last","first last"],[62,1,1,"coq:tacn.firstorder","firstorder"],[67,1,1,"coq:tacn.fix","fix"],[64,1,1,"coq:tacn.fold","fold"],[54,1,1,"coq:tacn.fresh","fresh"],[54,1,1,"coq:tacn.fun","fun"],[72,1,1,"coq:tacn.functional-induction","functional induction"],[72,1,1,"coq:tacn.functional-inversion","functional inversion"],[58,1,1,"coq:tacn.generalize","generalize"],[58,1,1,"coq:tacn.generalize-dependent","generalize dependent"],[58,1,1,"coq:tacn.generalize_eqs","generalize_eqs"],[58,1,1,"coq:tacn.generalize_eqs_vars","generalize_eqs_vars"],[57,1,1,"coq:tacn.generally-have","generally have"],[54,1,1,"coq:tacn.gfail","gfail"],[66,1,1,"coq:tacn.give_up","give_up"],[35,7,1,"coq:attr.global","global"],[54,1,1,"coq:tacn.guard","guard"],[54,1,1,"coq:tacn.has_evar","has_evar"],[57,1,1,"coq:tacn.have","have"],[3,1,1,"coq:tacn.head_of_constr","head_of_constr"],[64,1,1,"coq:tacn.hnf","hnf"],[54,1,1,"coq:tacn.idtac","idtac"],[55,1,1,"coq:tacn.if-then-else-(Ltac2)","if-then-else (Ltac2)"],[57,1,1,"coq:tacn.in","in"],[67,1,1,"coq:tacn.induction","induction"],[54,3,1,"coq:cmd.infoH","infoH"],[60,1,1,"coq:tacn.info_auto","info_auto"],[60,1,1,"coq:tacn.info_eauto","info_eauto"],[60,1,1,"coq:tacn.info_trivial","info_trivial"],[67,1,1,"coq:tacn.injection","injection"],[58,1,1,"coq:tacn.instantiate","instantiate"],[58,1,1,"coq:tacn.intro","intro"],[58,1,1,"coq:tacn.intros","intros"],[58,1,1,"coq:tacn.intros-until","intros until"],[62,1,1,"coq:tacn.intuition","intuition"],[67,1,1,"coq:tacn.inversion","inversion"],[67,1,1,"coq:tacn.inversion_clear","inversion_clear"],[67,1,1,"coq:tacn.inversion_sigma","inversion_sigma"],[54,1,1,"coq:tacn.is_cofix","is_cofix"],[54,1,1,"coq:tacn.is_const","is_const"],[54,1,1,"coq:tacn.is_constructor","is_constructor"],[54,1,1,"coq:tacn.is_evar","is_evar"],[54,1,1,"coq:tacn.is_fix","is_fix"],[54,1,1,"coq:tacn.is_ground","is_ground"],[54,1,1,"coq:tacn.is_ind","is_ind"],[54,1,1,"coq:tacn.is_proj","is_proj"],[54,1,1,"coq:tacn.is_var","is_var"],[58,1,1,"coq:tacn.lapply","lapply"],[58,0,1,"coq:exn.lapply-needs-a-non-dependent-product","lapply needs a non-dependent product"],[57,1,1,"coq:tacn.last","last"],[57,9,1,"coq:tacv.last-first","last first"],[64,1,1,"coq:tacn.lazy","lazy"],[55,1,1,"coq:tacn.lazy_match!","lazy_match!"],[55,1,1,"coq:tacn.lazy_match!-goal","lazy_match! goal"],[54,1,1,"coq:tacn.lazymatch","lazymatch"],[54,1,1,"coq:tacn.lazymatch-goal","lazymatch goal"],[67,1,1,"coq:tacn.left","left"],[54,1,1,"coq:tacn.let","let"],[5,1,1,"coq:tacn.lia","lia"],[35,7,1,"coq:attr.local","local"],[5,1,1,"coq:tacn.lra","lra"],[54,1,1,"coq:tacn.ltac-seq","ltac-seq"],[54,1,1,"coq:tacn.match","match"],[55,1,1,"coq:tacn.match-(Ltac2)","match (Ltac2)"],[54,1,1,"coq:tacn.match-goal","match goal"],[55,1,1,"coq:tacn.match!","match!"],[55,1,1,"coq:tacn.match!-goal","match! goal"],[13,7,1,"coq:attr.mode","mode"],[58,1,1,"coq:tacn.move","move"],[57,1,1,"coq:tacn.move-(ssreflect)","move (ssreflect)"],[55,1,1,"coq:tacn.multi_match!","multi_match!"],[55,1,1,"coq:tacn.multi_match!-goal","multi_match! goal"],[54,1,1,"coq:tacn.multimatch","multimatch"],[54,1,1,"coq:tacn.multimatch-goal","multimatch goal"],[58,1,1,"coq:tacn.native_cast_no_check","native_cast_no_check"],[64,1,1,"coq:tacn.native_compute","native_compute"],[5,1,1,"coq:tacn.nia","nia"],[4,7,1,"coq:attr.nonuniform","nonuniform"],[54,0,1,"coq:exn.not-a-cofix-definition","not a cofix definition"],[54,0,1,"coq:exn.not-a-constant","not a constant"],[54,0,1,"coq:exn.not-a-constructor","not a constructor"],[54,0,1,"coq:exn.not-a-fix-definition","not a fix definition"],[54,0,1,"coq:exn.not-a-primitive-projection","not a primitive projection"],[54,0,1,"coq:exn.not-an-(co)inductive-datatype","not an (co)inductive datatype"],[54,1,1,"coq:tacn.not_evar","not_evar"],[71,2,1,"coq:warn.notation-incompatible-prefix","notation-incompatible-prefix"],[60,1,1,"coq:tacn.now","now"],[64,1,1,"coq:tacn.now_show","now_show"],[5,1,1,"coq:tacn.nra","nra"],[7,1,1,"coq:tacn.nsatz","nsatz"],[7,1,1,"coq:tacn.nsatz_compute","nsatz_compute"],[54,1,1,"coq:tacn.numgoals","numgoals"],[54,1,1,"coq:tacn.once","once"],[54,1,1,"coq:tacn.only","only"],[54,1,1,"coq:tacn.optimize_heap","optimize_heap"],[57,1,1,"coq:tacn.over","over"],[71,0,1,"coq:exn.overflow-in-int63-literal-\u2018bigint\u2019","overflow in int63 literal \u2018bigint\u2019"],[64,1,1,"coq:tacn.pattern","pattern"],[58,1,1,"coq:tacn.pose","pose"],[57,1,1,"coq:tacn.pose-(ssreflect)","pose (ssreflect)"],[58,1,1,"coq:tacn.pose-proof","pose proof"],[71,2,1,"coq:warn.postfix-notation-not-level-1","postfix-notation-not-level-1"],[40,7,1,"coq:attr.private(matching)","private(matching)"],[9,7,1,"coq:attr.program","program"],[54,1,1,"coq:tacn.progress","progress"],[37,7,1,"coq:attr.projections(primitive)","projections(primitive)"],[11,1,1,"coq:tacn.protect_fv","protect_fv"],[5,1,1,"coq:tacn.psatz","psatz"],[59,0,1,"coq:exn.public-name-according-to-findlib,-for-example","public name according to findlib, for example"],[58,1,1,"coq:tacn.rapply","rapply"],[64,1,1,"coq:tacn.red","red"],[13,7,1,"coq:attr.refine","refine"],[58,1,1,"coq:tacn.refine","refine"],[64,1,1,"coq:tacn.reflexivity","reflexivity"],[58,1,1,"coq:tacn.remember","remember"],[58,1,1,"coq:tacn.rename","rename"],[54,1,1,"coq:tacn.repeat","repeat"],[64,1,1,"coq:tacn.replace","replace"],[54,1,1,"coq:tacn.reset-ltac-profile","reset ltac profile"],[54,1,1,"coq:tacn.restart_timer","restart_timer"],[4,7,1,"coq:attr.reversible","reversible"],[58,1,1,"coq:tacn.revert","revert"],[58,1,1,"coq:tacn.revert-dependent","revert dependent"],[66,1,1,"coq:tacn.revgoals","revgoals"],[64,1,1,"coq:tacn.rewrite","rewrite"],[57,1,1,"coq:tacn.rewrite-(ssreflect)","rewrite (ssreflect)"],[64,1,1,"coq:tacn.rewrite-*","rewrite *"],[3,1,1,"coq:tacn.rewrite_db","rewrite_db"],[3,1,1,"coq:tacn.rewrite_strat","rewrite_strat"],[67,1,1,"coq:tacn.right","right"],[11,1,1,"coq:tacn.ring","ring"],[11,1,1,"coq:tacn.ring_lookup","ring_lookup"],[11,1,1,"coq:tacn.ring_simplify","ring_simplify"],[62,1,1,"coq:tacn.rtauto","rtauto"],[58,1,1,"coq:tacn.set","set"],[57,1,1,"coq:tacn.set-(ssreflect)","set (ssreflect)"],[3,1,1,"coq:tacn.setoid_etransitivity","setoid_etransitivity"],[3,1,1,"coq:tacn.setoid_reflexivity","setoid_reflexivity"],[3,1,1,"coq:tacn.setoid_replace","setoid_replace"],[3,1,1,"coq:tacn.setoid_rewrite","setoid_rewrite"],[3,1,1,"coq:tacn.setoid_symmetry","setoid_symmetry"],[3,1,1,"coq:tacn.setoid_transitivity","setoid_transitivity"],[59,0,1,"coq:exn.shared-library-failed:-Coq-Error:-\u2018string\u2019-is-not-a-valid","shared library failed: Coq Error: \u2018string\u2019 is not a valid"],[66,1,1,"coq:tacn.shelve","shelve"],[66,1,1,"coq:tacn.shelve_unifiable","shelve_unifiable"],[54,1,1,"coq:tacn.show-ltac-profile","show ltac profile"],[64,1,1,"coq:tacn.simpl","simpl"],[58,1,1,"coq:tacn.simple-apply","simple apply"],[62,1,1,"coq:tacn.simple-congruence","simple congruence"],[67,1,1,"coq:tacn.simple-destruct","simple destruct"],[58,1,1,"coq:tacn.simple-eapply","simple eapply"],[67,1,1,"coq:tacn.simple-induction","simple induction"],[67,1,1,"coq:tacn.simple-injection","simple injection"],[67,1,1,"coq:tacn.simple-inversion","simple inversion"],[64,1,1,"coq:tacn.simple-subst","simple subst"],[67,1,1,"coq:tacn.simplify_eq","simplify_eq"],[72,1,1,"coq:tacn.soft-functional-induction","soft functional induction"],[54,1,1,"coq:tacn.solve","solve"],[66,1,1,"coq:tacn.solve_constraints","solve_constraints"],[58,1,1,"coq:tacn.specialize","specialize"],[58,1,1,"coq:tacn.specialize_eqs","specialize_eqs"],[67,1,1,"coq:tacn.split","split"],[27,1,1,"coq:tacn.split_Rabs","split_Rabs"],[27,1,1,"coq:tacn.split_Rmult","split_Rmult"],[54,1,1,"coq:tacn.start-ltac-profiling","start ltac profiling"],[64,1,1,"coq:tacn.stepl","stepl"],[64,1,1,"coq:tacn.stepr","stepr"],[54,1,1,"coq:tacn.stop-ltac-profiling","stop ltac profiling"],[64,1,1,"coq:tacn.subst","subst"],[64,1,1,"coq:tacn.substitute","substitute"],[57,1,1,"coq:tacn.suff","suff"],[57,1,1,"coq:tacn.suffices","suffices"],[66,1,1,"coq:tacn.swap","swap"],[64,1,1,"coq:tacn.symmetry","symmetry"],[62,1,1,"coq:tacn.tauto","tauto"],[34,0,1,"coq:exn.template-and-polymorphism-not-compatible","template and polymorphism not compatible"],[54,1,1,"coq:tacn.time","time"],[54,1,1,"coq:tacn.time_constr","time_constr"],[54,1,1,"coq:tacn.timeout","timeout"],[64,1,1,"coq:tacn.transitivity","transitivity"],[66,1,1,"coq:tacn.transparent_abstract","transparent_abstract"],[60,1,1,"coq:tacn.trivial","trivial"],[54,1,1,"coq:tacn.try","try"],[54,1,1,"coq:tacn.tryif","tryif"],[54,1,1,"coq:tacn.type-of","type of"],[54,1,1,"coq:tacn.type_term","type_term"],[13,1,1,"coq:tacn.typeclasses-eauto","typeclasses eauto"],[57,1,1,"coq:tacn.under","under"],[64,1,1,"coq:tacn.unfold","unfold"],[54,1,1,"coq:tacn.unify","unify"],[14,7,1,"coq:attr.universes(cumulative)","universes(cumulative)"],[14,7,1,"coq:attr.universes(polymorphic)","universes(polymorphic)"],[34,7,1,"coq:attr.universes(template)","universes(template)"],[57,1,1,"coq:tacn.unlock","unlock"],[66,1,1,"coq:tacn.unshelve","unshelve"],[66,7,1,"coq:attr.using","using"],[58,1,1,"coq:tacn.vm_cast_no_check","vm_cast_no_check"],[64,1,1,"coq:tacn.vm_compute","vm_compute"],[74,7,1,"coq:attr.warn","warn"],[29,7,1,"coq:attr.warning","warning"],[29,7,1,"coq:attr.warnings","warnings"],[64,1,1,"coq:tacn.with_strategy","with_strategy"],[57,1,1,"coq:tacn.without-loss","without loss"],[5,1,1,"coq:tacn.wlia","wlia"],[57,1,1,"coq:tacn.wlog","wlog"],[5,1,1,"coq:tacn.wlra_Q","wlra_Q"],[5,1,1,"coq:tacn.wnia","wnia"],[5,1,1,"coq:tacn.wnra_Q","wnra_Q"],[5,1,1,"coq:tacn.wpsatz_Q","wpsatz_Q"],[5,1,1,"coq:tacn.wpsatz_Z","wpsatz_Z"],[5,1,1,"coq:tacn.wsos_Q","wsos_Q"],[5,1,1,"coq:tacn.wsos_Z","wsos_Z"],[5,1,1,"coq:tacn.xlia","xlia"],[5,1,1,"coq:tacn.xlra_Q","xlra_Q"],[5,1,1,"coq:tacn.xlra_R","xlra_R"],[5,1,1,"coq:tacn.xnia","xnia"],[5,1,1,"coq:tacn.xnra_Q","xnra_Q"],[5,1,1,"coq:tacn.xnra_R","xnra_R"],[5,1,1,"coq:tacn.xpsatz_Q","xpsatz_Q"],[5,1,1,"coq:tacn.xpsatz_R","xpsatz_R"],[5,1,1,"coq:tacn.xpsatz_Z","xpsatz_Z"],[5,1,1,"coq:tacn.xsos_Q","xsos_Q"],[5,1,1,"coq:tacn.xsos_R","xsos_R"],[5,1,1,"coq:tacn.xsos_Z","xsos_Z"],[5,1,1,"coq:tacn.zify","zify"],[5,1,1,"coq:tacn.zify_elim_let","zify_elim_let"],[5,1,1,"coq:tacn.zify_iter_let","zify_iter_let"],[5,1,1,"coq:tacn.zify_iter_specs","zify_iter_specs"],[5,1,1,"coq:tacn.zify_op","zify_op"],[5,1,1,"coq:tacn.zify_saturate","zify_saturate"],[66,1,1,"coq:tacn.{","{"],[54,1,1,"coq:tacn.||-(first-tactic-making-progress)","|| (first tactic making progress)"],[66,1,1,"coq:tacn.}","}"],[4,0,1,"coq:exn.\u2018coercion_class\u2019-must-be-a-transparent-constant","\u2018coercion_class\u2019 must be a transparent constant"],[37,0,1,"coq:exn.\u2018ident\u2019-already-exists","\u2018ident\u2019 already exists"],[37,2,1,"coq:warn.\u2018ident\u2019-cannot-be-defined","\u2018ident\u2019 cannot be defined"],[37,2,1,"coq:warn.\u2018ident\u2019-cannot-be-defined-because-it-is-informative-and-\u2018ident\u2019-is-not","\u2018ident\u2019 cannot be defined because it is informative and \u2018ident\u2019 is not"],[37,2,1,"coq:warn.\u2018ident\u2019-cannot-be-defined-because-the-projection-\u2018ident\u2019-was-not-defined","\u2018ident\u2019 cannot be defined because the projection \u2018ident\u2019 was not defined"],[13,2,1,"coq:warn.\u2018ident\u2019-is-already-declared-as-a-typeclass","\u2018ident\u2019 is already declared as a typeclass"],[58,0,1,"coq:exn.\u2018ident\u2019-is-already-used","\u2018ident\u2019 is already used"],[66,2,1,"coq:warn.\u2018ident\u2019-is-both-name-of-a-Collection-and-Variable,-Collection-\u2018ident\u2019-takes-precedence-over-Variable","\u2018ident\u2019 is both name of a Collection and Variable, Collection \u2018ident\u2019 takes precedence over Variable"],[58,0,1,"coq:exn.\u2018ident\u2019-is-not-a-local-definition","\u2018ident\u2019 is not a local definition"],[67,0,1,"coq:exn.\u2018ident\u2019-is-not-an-equality-of-\u03a3-types","\u2018ident\u2019 is not an equality of \u03a3 types"],[64,0,1,"coq:exn.\u2018ident\u2019-is-opaque","\u2018ident\u2019 is opaque"],[58,0,1,"coq:exn.\u2018ident\u2019-is-used-in-the-conclusion","\u2018ident\u2019 is used in the conclusion"],[58,0,1,"coq:exn.\u2018ident\u2019-is-used-in-the-hypothesis-\u2018ident\u2019","\u2018ident\u2019 is used in the hypothesis \u2018ident\u2019"],[66,2,1,"coq:warn.\u2018ident\u2019-was-already-a-defined-Variable,-the-name-\u2018ident\u2019-will-refer-to-Collection-when-executing-\"Proof-using\"-command","\u2018ident\u2019 was already a defined Variable, the name \u2018ident\u2019 will refer to Collection when executing "Proof using" command"],[60,0,1,"coq:exn.\u2018qualid\u2019-cannot-be-used-as-a-hint","\u2018qualid\u2019 cannot be used as a hint"],[64,0,1,"coq:exn.\u2018qualid\u2019-does-not-occur","\u2018qualid\u2019 does not occur"],[4,2,1,"coq:warn.\u2018qualid\u2019-does-not-respect-the-uniform-inheritance-condition","\u2018qualid\u2019 does not respect the uniform inheritance condition"],[4,0,1,"coq:exn.\u2018qualid\u2019-is-already-a-coercion","\u2018qualid\u2019 is already a coercion"],[71,0,1,"coq:exn.\u2018qualid\u2019-is-bound-to-a-notation-that-does-not-denote-a-reference","\u2018qualid\u2019 is bound to a notation that does not denote a reference"],[4,0,1,"coq:exn.\u2018qualid\u2019-is-not-a-function","\u2018qualid\u2019 is not a function"],[35,0,1,"coq:exn.\u2018qualid\u2019-is-not-a-module","\u2018qualid\u2019 is not a module"],[60,0,1,"coq:exn.\u2018qualid\u2019-is-not-an-inductive-type","\u2018qualid\u2019 is not an inductive type"],[59,0,1,"coq:exn.\u2018qualid\u2019-not-a-defined-object","\u2018qualid\u2019 not a defined object"],[4,0,1,"coq:exn.\u2018qualid\u2019-not-declared","\u2018qualid\u2019 not declared"],[71,0,1,"coq:exn.\u2018qualid\u2019-was-already-mapped-to-\u2018qualid\u2019-and-cannot-be-remapped-to-\u2018qualid\u2019","\u2018qualid\u2019 was already mapped to \u2018qualid\u2019 and cannot be remapped to \u2018qualid\u2019"],[74,2,1,"coq:warn.\u2018string\u2019","\u2018string\u2019"],[71,0,1,"coq:exn.\u2018type\u2019-is-not-an-inductive-type","\u2018type\u2019 is not an inductive type"],[71,2,1,"coq:warn.\u2018type\u2019-was-already-mapped-to-\u2018type\u2019,-mapping-it-also-to-\u2018type\u2019-might-yield-ill-typed-terms-when-using-the-notation","\u2018type\u2019 was already mapped to \u2018type\u2019, mapping it also to \u2018type\u2019 might yield ill typed terms when using the notation"],[54,1,1,"coq:tacn.\u2026-:-\u2026-(goal-selector)","\u2026 : \u2026 (goal selector)"],[57,1,1,"coq:tacn.\u2026-:-\u2026-(ssreflect)","\u2026 : \u2026 (ssreflect)"]],""All" is a predefined collection containing all variables":[[66,0,1,"coq:exn.\"All\"-is-a-predefined-collection-containing-all-variables.-It-can't-be-redefined"," It can't be redefined"]],"..":[[4,2,1,"coq:warn....-is-not-definitionally-an-identity-function"," is not definitionally an identity function"]],"Argument \u2018name\u2019 is a trailing implicit, so it can't be declared non maximal":[[44,0,1,"coq:exn.Argument-\u2018name\u2019-is-a-trailing-implicit,-so-it-can't-be-declared-non-maximal.-Please-use-{-}-instead-of-[-]"," Please use { } instead of [ ]"]],"Cannot infer a term for this placeholder":[[44,0,1,"coq:exn.Cannot-infer-a-term-for-this-placeholder.-(Casual-use-of-implicit-arguments)"," (Casual use of implicit arguments)"],[58,0,1,"coq:exn.Cannot-infer-a-term-for-this-placeholder.-(refine)"," (refine)"]],"Compiled library \u2018ident\u2019":[[59,0,1,"coq:exn.Compiled-library-\u2018ident\u2019.vo-makes-inconsistent-assumptions-over-library-\u2018qualid\u2019","vo makes inconsistent assumptions over library \u2018qualid\u2019"]],"Duplicate clear of H":[[57,2,1,"coq:warn.Duplicate-clear-of-H.-Use-{-}H-instead-of-{-H-}H"," Use { }H instead of { H }H"]],"File ... found twice in ..":[[59,2,1,"coq:warn.File-...-found-twice-in-...",""]],"Goal is solvable by congruence but some arguments are missing":[[62,0,1,"coq:exn.Goal-is-solvable-by-congruence-but-some-arguments-are-missing.-Try-congruence-with-\u2018term\u2019\u2026\u2018term\u2019,-replacing-metavariables-by-arbitrary-terms"," Try congruence with \u2018term\u2019\u2026\u2018term\u2019, replacing metavariables by arbitrary terms"]],"Library File (transitively required) \u2018qualid\u2019 is deprecated since \u2018string\u2019. \u2018string\u2019":[[74,2,1,"coq:warn.Library-File-(transitively-required)-\u2018qualid\u2019-is-deprecated-since-\u2018string\u2019.-\u2018string\u2019.-Use-\u2018qualid\u2019-instead"," Use \u2018qualid\u2019 instead"]],"Library File \u2018qualid\u2019 is deprecated since \u2018string\u2019. \u2018string\u2019":[[74,2,1,"coq:warn.Library-File-\u2018qualid\u2019-is-deprecated-since-\u2018string\u2019.-\u2018string\u2019.-Use-\u2018qualid\u2019-instead"," Use \u2018qualid\u2019 instead"]],"Ltac Profiler encountered an invalid stack (no self node)":[[54,2,1,"coq:warn.Ltac-Profiler-encountered-an-invalid-stack-(no-self-node).-This-can-happen-if-you-reset-the-profile-during-tactic-execution"," This can happen if you reset the profile during tactic execution"]],"Ltac2 alias \u2018qualid\u2019 is deprecated since \u2018string\u2019":[[74,2,1,"coq:warn.Ltac2-alias-\u2018qualid\u2019-is-deprecated-since-\u2018string\u2019.-\u2018string\u2019"," \u2018string\u2019"]],"Ltac2 constructor \u2018qualid\u2019 is deprecated since \u2018string\u2019":[[74,2,1,"coq:warn.Ltac2-constructor-\u2018qualid\u2019-is-deprecated-since-\u2018string\u2019.-\u2018string\u2019"," \u2018string\u2019"]],"Ltac2 definition \u2018qualid\u2019 is deprecated since \u2018string\u2019":[[74,2,1,"coq:warn.Ltac2-definition-\u2018qualid\u2019-is-deprecated-since-\u2018string\u2019.-\u2018string\u2019"," \u2018string\u2019"]],"Ltac2 notation \u2018ltac2_scope\u2019\u2026\u2018ltac2_scope\u2019 is deprecated since \u2018string\u2019":[[74,2,1,"coq:warn.Ltac2-notation-\u2018ltac2_scope\u2019\u2026\u2018ltac2_scope\u2019-is-deprecated-since-\u2018string\u2019.-\u2018string\u2019"," \u2018string\u2019"]],"Nested proofs are discouraged and not allowed by default. This error probably means that you forgot to close the last "Proof." with "Qed." or "Defined."":[[32,0,1,"coq:exn.Nested-proofs-are-discouraged-and-not-allowed-by-default.-This-error-probably-means-that-you-forgot-to-close-the-last-\"Proof.\"-with-\"Qed.\"-or-\"Defined.\".-If-you-really-intended-to-use-nested-proofs,-you-can-do-so-by-turning-the-\"Nested-Proofs-Allowed\"-flag-on"," If you really intended to use nested proofs, you can do so by turning the "Nested Proofs Allowed" flag on"]],"New coercion path ... is ambiguous with existing ..":[[4,2,1,"coq:warn.New-coercion-path-...-is-ambiguous-with-existing-...",""]],"No information can be deduced from this equality and the injectivity of constructors. This may be because the terms are convertible, or due to pattern matching restrictions in the sort Prop":[[67,0,1,"coq:exn.No-information-can-be-deduced-from-this-equality-and-the-injectivity-of-constructors.-This-may-be-because-the-terms-are-convertible,-or-due-to-pattern-matching-restrictions-in-the-sort-Prop.-You-can-try-to-use-option-Set-Keep-Proof-Equalities"," You can try to use option Set Keep Proof Equalities"]],"No such bound variable \u2018ident\u2019 (possible names are: \u2018ident\u2019 ..":[[58,0,1,"coq:exn.No-such-bound-variable-\u2018ident\u2019-(possible-names-are:-\u2018ident\u2019-...)",")"]],"No such goal":[[54,0,1,"coq:exn.No-such-goal.-(Goal-selector)"," (Goal selector)"],[54,0,1,"coq:exn.No-such-goal.-(fail)"," (fail)"],[66,0,1,"coq:exn.No-such-goal.-Focus-next-goal-with-bullet-\u2018bullet\u2019"," Focus next goal with bullet \u2018bullet\u2019"],[66,0,1,"coq:exn.No-such-goal.-Try-unfocusing-with-}"," Try unfocusing with }"]],"Notation \u2018string\u2019 is deprecated since \u2018string\u2019. \u2018string\u2019":[[74,2,1,"coq:warn.Notation-\u2018string\u2019-is-deprecated-since-\u2018string\u2019.-\u2018string\u2019.-Use-\u2018qualid\u2019-instead"," Use \u2018qualid\u2019 instead"]],"Proof is not complete":[[66,0,1,"coq:exn.Proof-is-not-complete.-(abstract)"," (abstract)"],[58,0,1,"coq:exn.Proof-is-not-complete.-(assert)"," (assert)"]],"Require inside a module is deprecated and strongly discouraged":[[59,2,1,"coq:warn.Require-inside-a-module-is-deprecated-and-strongly-discouraged.-You-can-Require-a-module-at-toplevel-and-optionally-Import-it-inside-another-one"," You can Require a module at toplevel and optionally Import it inside another one"]],"Required library \u2018qualid\u2019 matches several files in path (found file.vo, file.vo, ..":[[59,0,1,"coq:exn.Required-library-\u2018qualid\u2019-matches-several-files-in-path-(found-file.vo,-file.vo,-...)",")"]],"SSReflect: cannot obtain new equations out of ..":[[57,2,1,"coq:warn.SSReflect:-cannot-obtain-new-equations-out-of-...",""]],"Tactic Notation \u2018qualid\u2019 is deprecated since \u2018string\u2019":[[74,2,1,"coq:warn.Tactic-Notation-\u2018qualid\u2019-is-deprecated-since-\u2018string\u2019.-\u2018string\u2019"," \u2018string\u2019"]],"Tactic \u2018qualid\u2019 is deprecated since \u2018string\u2019":[[74,2,1,"coq:warn.Tactic-\u2018qualid\u2019-is-deprecated-since-\u2018string\u2019.-\u2018string\u2019"," \u2018string\u2019"]],"The constant \u2018number\u2019 is not a binary64 floating-point value. A closest value \u2018number\u2019 will be used and unambiguously printed \u2018number\u2019":[[27,2,1,"coq:warn.The-constant-\u2018number\u2019-is-not-a-binary64-floating-point-value.-A-closest-value-\u2018number\u2019-will-be-used-and-unambiguously-printed-\u2018number\u2019.-[inexact-float,parsing]"," [inexact-float,parsing]"]],"The file \u2018ident\u2019":[[59,0,1,"coq:exn.The-file-\u2018ident\u2019.vo-contains-library-\u2018qualid\u2019-and-not-library-\u2018qualid\u2019","vo contains library \u2018qualid\u2019 and not library \u2018qualid\u2019"]],"The relation \u2018ident\u2019 is not a declared reflexive relation. Maybe you need to require the Stdlib.Classes":[[64,0,1,"coq:exn.The-relation-\u2018ident\u2019-is-not-a-declared-reflexive-relation.-Maybe-you-need-to-require-the-Stdlib.Classes.RelationClasses-library","RelationClasses library"]],"The relation \u2018ident\u2019 is not a declared symmetric relation. Maybe you need to require the Stdlib.Classes":[[64,0,1,"coq:exn.The-relation-\u2018ident\u2019-is-not-a-declared-symmetric-relation.-Maybe-you-need-to-require-the-Stdlib.Classes.RelationClasses-library","RelationClasses library"]],"The relation \u2018ident\u2019 is not a declared transitive relation. Maybe you need to require the Stdlib.Classes":[[64,0,1,"coq:exn.The-relation-\u2018ident\u2019-is-not-a-declared-transitive-relation.-Maybe-you-need-to-require-the-Stdlib.Classes.RelationClasses-library","RelationClasses library"]],"This command is just asserting the names of arguments of \u2018qualid\u2019. If this is what you want, add ': assert' to silence the warning. If you want to clear implicit arguments, add ': clear implicits'":[[41,2,1,"coq:warn.This-command-is-just-asserting-the-names-of-arguments-of-\u2018qualid\u2019.-If-this-is-what-you-want,-add-':-assert'-to-silence-the-warning.-If-you-want-to-clear-implicit-arguments,-add-':-clear-implicits'.-If-you-want-to-clear-notation-scopes,-add-':-clear-scopes'"," If you want to clear notation scopes, add ': clear scopes'"]],"This hint is not local but depends on a section variable":[[60,2,1,"coq:warn.This-hint-is-not-local-but-depends-on-a-section-variable.-It-will-disappear-when-the-section-is-closed"," It will disappear when the section is closed"]],"Type of \u2018qualid\u2019 seems incompatible with the type of \u2018qualid\u2019. Expected type is: \u2018type\u2019 instead of \u2018type\u2019":[[71,2,1,"coq:warn.Type-of-\u2018qualid\u2019-seems-incompatible-with-the-type-of-\u2018qualid\u2019.-Expected-type-is:-\u2018type\u2019-instead-of-\u2018type\u2019.-This-might-yield-ill-typed-terms-when-using-the-notation"," This might yield ill typed terms when using the notation"]],"Unable to apply lemma of type "..." on hypothesis of type "..":[[58,0,1,"coq:exn.Unable-to-apply-lemma-of-type-\"...\"-on-hypothesis-of-type-\"...\"","""]],"Unused variable \u2018ident\u2019 might be a misspelled constructor. Use _ or _\u2018ident\u2019 to silence this warning":[[46,2,1,"coq:warn.Unused-variable-\u2018ident\u2019-might-be-a-misspelled-constructor.-Use-_-or-_\u2018ident\u2019-to-silence-this-warning.",""]],"\u2018ident\u2019 already exists":[[28,0,1,"coq:exn.\u2018ident\u2019-already-exists.-(Axiom)"," (Axiom)"],[32,0,1,"coq:exn.\u2018ident\u2019-already-exists.-(Definition)"," (Definition)"],[32,0,1,"coq:exn.\u2018ident\u2019-already-exists.-(Theorem)"," (Theorem)"]],"\u2018qualid\u2019 should go from Byte.byte, (list Byte.byte), or PrimString":[[71,0,1,"coq:exn.\u2018qualid\u2019-should-go-from-Byte.byte,-(list-Byte.byte),-or-PrimString.string-to-\u2018type\u2019-or-(option-\u2018type\u2019)","string to \u2018type\u2019 or (option \u2018type\u2019)"]],"\u2018qualid\u2019 should go from Number.int to \u2018type\u2019 or (option \u2018type\u2019). Instead of Number.int, the types Number.uint or Z or PrimInt63.pos_neg_int63 or PrimFloat.float or Number":[[71,0,1,"coq:exn.\u2018qualid\u2019-should-go-from-Number.int-to-\u2018type\u2019-or-(option-\u2018type\u2019).-Instead-of-Number.int,-the-types-Number.uint-or-Z-or-PrimInt63.pos_neg_int63-or-PrimFloat.float-or-Number.number-could-be-used-(you-may-need-to-require-BinNums-or-Number-or-PrimInt63-or-PrimFloat-first)","number could be used (you may need to require BinNums or Number or PrimInt63 or PrimFloat first)"]],"\u2018qualid\u2019 should go from \u2018type\u2019 to Number.int or (option Number.int). Instead of Number.int, the types Number.uint or Z or PrimInt63.pos_neg_int63 or Number":[[71,0,1,"coq:exn.\u2018qualid\u2019-should-go-from-\u2018type\u2019-to-Number.int-or-(option-Number.int).-Instead-of-Number.int,-the-types-Number.uint-or-Z-or-PrimInt63.pos_neg_int63-or-Number.number-could-be-used-(you-may-need-to-require-BinNums-or-Number-or-PrimInt63-first)","number could be used (you may need to require BinNums or Number or PrimInt63 first)"]],"\u2018qualid\u2019 should go from \u2018type\u2019 to T or (option T), where T is either Byte.byte, (list Byte.byte), or PrimString":[[71,0,1,"coq:exn.\u2018qualid\u2019-should-go-from-\u2018type\u2019-to-T-or-(option-T),-where-T-is-either-Byte.byte,-(list-Byte.byte),-or-PrimString.string","string"]],"\u2018string\u2019 cannot be interpreted as a known notation in \u2018ident\u2019 entry":[[71,0,1,"coq:exn.\u2018string\u2019-cannot-be-interpreted-as-a-known-notation-in-\u2018ident\u2019-entry.-Make-sure-that-symbols-are-surrounded-by-spaces-and-that-holes-are-explicitly-denoted-by-\"_\""," Make sure that symbols are surrounded by spaces and that holes are explicitly denoted by "_""]],"\u2018string\u2019 cannot be interpreted as a known notation":[[71,0,1,"coq:exn.\u2018string\u2019-cannot-be-interpreted-as-a-known-notation.-Make-sure-that-symbols-are-surrounded-by-spaces-and-that-holes-are-explicitly-denoted-by-\"_\""," Make sure that symbols are surrounded by spaces and that holes are explicitly denoted by "_""]],"package-name":[[59,0,1,"coq:exn.package-name.foo-and-not-foo_plugin","foo and not foo_plugin"]],"plugin name anymore":[[59,0,1,"coq:exn.plugin-name-anymore.-Plugins-should-be-loaded-using-their"," Plugins should be loaded using their"]]},objnames:{"0":["coq","exn","Coq exn"],"1":["coq","tacn","Coq tacn"],"2":["coq","warn","Coq warn"],"3":["coq","cmd","Coq cmd"],"4":["coq","flag","Coq flag"],"5":["coq","thm","Coq thm"],"6":["coq","opt","Coq opt"],"7":["coq","attr","Coq attr"],"8":["coq","table","Coq table"],"9":["coq","tacv","Coq tacv"]},objtypes:{"0":"coq:exn","1":"coq:tacn","2":"coq:warn","3":"coq:cmd","4":"coq:flag","5":"coq:thm","6":"coq:opt","7":"coq:attr","8":"coq:table","9":"coq:tacv"},terms:{"0":[2,3,4,5,7,8,9,10,11,12,13,14,25,26,27,28,29,30,31,34,35,36,37,41,43,44,46,50,51,52,53,54,55,57,58,59,60,62,64,66,67,71,72,74,75,77],"00":53,"000":[17,53],"0000000000000002":27,"00075471":77,"00076024":77,"00076039":77,"001":64,"001u":64,"002":54,"005":54,"00816703":77,"01":[17,53,64],"012":54,"019":53,"02":[17,29,53,77],"02451322":77,"026":53,"027":53,"028":53,"02e":[17,29],"03":[8,17,53],"032":54,"0380":17,"03ff":17,"04":53,"05":17,"0515":77,"0530":77,"05ef":17,"06":[17,24,53,77],"068":53,"069":53,"07":[17,77],"08":[17,77],"09":17,"0beta":25,"0m00":53,"0m03":53,"0m04":53,"0s":71,"0x":29,"0x2a":17,"0xap12":29,"0xb":17,"1":[0,1,2,3,4,5,6,7,8,9,10,11,12,13,14,15,16,18,19,20,21,22,23,25,26,27,28,29,30,31,32,33,34,35,36,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,68,69,70,71,72,73,74,75,76,77],"10":[2,5,24,25,29,31,52,54,57,59,60,64,71,74,77],"100":[17,54,60,64,71],"1000":[62,64],"100000":29,"1000000":29,"1000000000000000000000000000000000":29,"1000000000000000000000000000000001":29,"10002":17,"10008":17,"10012":17,"10014":17,"10017":17,"10019":17,"10022":17,"10049":17,"10053":17,"10059":17,"10061":17,"1007":77,"10076":17,"10085":17,"10088":17,"10095":17,"101":14,"10108":17,"10110":17,"10111":17,"10112":17,"10117":17,"10156":17,"10167":17,"10173":17,"10180":17,"10185":17,"10202":17,"10205":17,"10215":17,"1024":2,"10245":17,"10277":17,"10289":17,"10291":17,"102e":17,"102u":64,"10301":17,"10302":17,"10305":17,"10318":17,"10324":17,"10331":17,"10336":17,"10343":17,"10360":17,"10361":17,"10366":17,"10390":17,"10399":17,"104":77,"10400":17,"10407":17,"10430":17,"10439":17,"10441":17,"10445":17,"10471":17,"10476":17,"10486":17,"10489":17,"10494":17,"105":17,"10577":17,"10592":17,"10614":17,"10651":17,"10657":17,"10664":17,"10728":17,"10731":17,"10739":17,"10747":17,"10750":17,"10757":17,"10758":17,"10760":17,"10762":17,"10765":17,"10772":17,"10774":17,"10796":17,"10803":17,"10806":17,"10811":17,"10812":17,"10816":17,"10824":17,"10827":17,"10832":17,"10842":17,"10852":17,"10858":17,"1088":77,"10891":17,"10894":17,"10895":17,"10897":17,"10899":17,"10904":17,"10912":17,"10932":17,"10947":17,"10956":17,"10963":17,"10965":17,"10966":17,"10970":17,"10971":17,"10985":17,"10988":17,"10996":17,"10997":17,"10998":17,"11":[2,24,25,34,53,57,60],"110":60,"11000":17,"11011":17,"11014":17,"11018":17,"11024":17,"11025":17,"11030":17,"11033":17,"11039":17,"11048":17,"11052":17,"11058":17,"11063":17,"11068":17,"11069":17,"11070":17,"11080":17,"11081":17,"11090":17,"11091":17,"11098":17,"11099":17,"11102":17,"11113":17,"11114":17,"11120":17,"11121":17,"11123":17,"11127":17,"11128":17,"11131":17,"11132":17,"11136":17,"11162":17,"11164":17,"11172":17,"11183":17,"11185":17,"11187":17,"11191":17,"11203":17,"11227":17,"11231":17,"11233":17,"11235":17,"11237":17,"11240":17,"11241":17,"11242":17,"11245":17,"11249":17,"11254":17,"11255":17,"11258":17,"11261":17,"11263":17,"11270":17,"11276":17,"11277":17,"11280":17,"11288":17,"11295":17,"113":[17,64],"11301":17,"11302":17,"11311":17,"11314":17,"11329":17,"11331":17,"11335":17,"11337":17,"11350":17,"11353":17,"11357":17,"11360":17,"11361":17,"11362":17,"11368":17,"11370":17,"11394":17,"11396":17,"11400":17,"11402":17,"11404":17,"11409":17,"11414":17,"11415":17,"11422":17,"11423":17,"11428":17,"11429":17,"11430":17,"11436":17,"11447":17,"1145":77,"11471":17,"11474":17,"11486":17,"11503":17,"11504":17,"11506":17,"11522":17,"11523":17,"11530":17,"11534":17,"11537":17,"11546":17,"11579":17,"1158":77,"11585":17,"11586":17,"11589":17,"11590":17,"11595":17,"11600":17,"11601":17,"11602":17,"11604":17,"11606":17,"11617":17,"11618":17,"11631":17,"11650":17,"11663":17,"11665":17,"11686":17,"11689":17,"117":77,"11705":17,"11718":17,"11720":17,"11725":17,"11727":17,"11740":17,"11741":17,"11742":17,"11746":17,"11755":17,"11760":17,"11761":17,"11766":17,"11783":17,"11795":17,"11797":17,"118":10,"11811":17,"11812":17,"11816":17,"11828":17,"11841":17,"11848":17,"11851":17,"11859":17,"11866":17,"11869":17,"11871":17,"11877":17,"11880":17,"11882":17,"11883":17,"11885":17,"11890":17,"11891":17,"11903":17,"11905":17,"11906":17,"11909":17,"11913":17,"11914":17,"11943":17,"11944":17,"11946":17,"11948":17,"11957":17,"11958":17,"11960":17,"11961":17,"11962":17,"11963":17,"11970":17,"11972":17,"11976":17,"11981":17,"11986":17,"11988":17,"11992":17,"12":[11,25,29,53,54,57,58,60,71],"120":[51,71],"12001":17,"12005":17,"12006":17,"12008":17,"12011":17,"12014":17,"12015":17,"12018":17,"12023":17,"12026":17,"12027":17,"12031":17,"12033":17,"12034":17,"12035":17,"12037":17,"12044":17,"12045":17,"12060":17,"12068":17,"12070":17,"12073":17,"12076":17,"12091":17,"12093":17,"12094":17,"12096":17,"12097":17,"12099":17,"12103":17,"12106":17,"12109":17,"12116":17,"12120":17,"12121":17,"12126":17,"12129":17,"12139":17,"12146":17,"12148":17,"12150":17,"12152":17,"12157":17,"12159":17,"12162":17,"12163":17,"12172":17,"12186":17,"12196":17,"12197":17,"12200":64,"12210":17,"12211":17,"12213":17,"12218":17,"12223":17,"12224":17,"12228":17,"12233":17,"12234":17,"12237":17,"12239":17,"12240":17,"12246":17,"12253":17,"12254":17,"12255":17,"12256":17,"12257":17,"12258":17,"12263":17,"12266":17,"12286":17,"12287":17,"12288":17,"12295":17,"12296":17,"123":71,"12317":17,"12322":17,"12323":17,"12324":17,"12326":17,"12330":17,"12332":17,"12348":17,"12358":17,"12365":17,"12366":17,"12368":17,"12387":17,"12388":17,"12389":17,"12399":17,"12411":17,"12414":17,"12418":17,"12420":17,"12422":17,"12423":[17,54],"12425":17,"12454":17,"12467":17,"12479":17,"12483":17,"12484":17,"12513":17,"12516":17,"12521":17,"12523":17,"12525":17,"12537":17,"12541":17,"12552":17,"12556":17,"12562":17,"12567":17,"12571":17,"12572":17,"12575":17,"12582":17,"12583":17,"12586":17,"12594":17,"12595":17,"126":[53,54],"12613":17,"12647":17,"12648":17,"12653":17,"12677":17,"12678":17,"12682":17,"12683":17,"12685":17,"12707":17,"12708":17,"12716":17,"12738":17,"12752":17,"12754":17,"12755":17,"12756":17,"12762":17,"12765":17,"12768":17,"12770":17,"12772":17,"12773":17,"12775":17,"12777":17,"12787":17,"12793":17,"12794":17,"12799":17,"128":[2,54],"12801":17,"12803":17,"12806":17,"1281":77,"12813":17,"12816":17,"12827":17,"12837":17,"12845":17,"12846":17,"12847":17,"12857":17,"12860":17,"12861":17,"12862":17,"12871":17,"12874":17,"128mb":51,"128u":53,"12908":17,"12946":17,"12948":17,"12950":17,"12960":17,"12965":17,"12972":17,"12975":17,"12979":17,"12984":17,"12986":17,"12992":17,"13":[24,25,51,54,57,77],"13004":17,"13007":17,"13011":17,"13016":17,"13018":17,"13026":17,"13028":17,"13040":17,"13062":17,"13063":17,"13067":17,"13071":17,"13078":17,"13080":17,"13092":17,"13096":17,"13106":17,"13139":17,"13145":17,"13150":17,"13155":17,"13157":17,"13165":17,"13166":17,"13183":17,"13188":17,"13189":17,"13202":17,"13216":17,"13217":17,"13232":17,"13235":17,"13236":17,"13237":17,"13244":17,"13247":17,"13255":17,"13265":17,"13266":17,"13278":17,"13287":17,"13288":17,"13290":17,"13296":17,"13298":17,"13301":17,"13303":17,"13307":17,"13312":17,"13317":17,"13330":17,"13331":17,"13336":17,"13337":17,"13339":17,"13344":17,"13345":17,"13349":17,"13351":17,"13352":17,"13354":17,"13356":17,"13363":17,"13365":17,"13373":17,"13376":17,"13381":17,"13383":17,"13384":17,"13386":17,"13387":17,"13388":17,"13394":17,"13403":17,"13405":17,"13408":17,"13413":17,"13415":17,"13417":17,"13428":17,"13432":17,"13436":17,"13442":17,"13448":17,"13456":17,"13458":17,"13459":17,"13460":17,"13468":17,"13469":17,"1347":17,"13473":17,"13480":17,"13484":17,"13490":17,"13495":17,"135":77,"13501":17,"13509":17,"13512":17,"13517":17,"13519":17,"13541":17,"13550":17,"13556":17,"13559":17,"13562":17,"13563":17,"13566":17,"13568":17,"13579":17,"13581":17,"13582":17,"13586":17,"13589":17,"13617":17,"13618":17,"1362":17,"13624":17,"13654":17,"13671":17,"13696":17,"13699":17,"136u":53,"137":27,"13702":17,"13715":17,"13724":17,"13725":17,"13727":17,"13741":17,"13758":17,"13759":17,"13760":17,"13761":17,"13762":17,"13763":17,"13764":17,"13774":17,"13778":17,"13781":17,"13783":17,"13804":17,"13810":17,"13812":17,"13822":17,"13830":17,"13837":17,"1384":24,"13840":17,"13842":17,"13849":17,"13852":17,"13853":17,"13859":17,"1386":24,"13867":17,"1387":24,"13870":17,"13871":17,"13876":17,"13882":17,"13885":17,"13895":17,"13909":17,"13911":17,"13912":17,"13914":17,"13920":17,"13927":17,"13939":17,"1394":24,"13942":17,"13952":17,"13955":17,"13964":17,"13965":17,"13966":17,"13967":17,"13969":17,"13976":17,"13977":17,"13986":17,"13996":17,"13997":17,"13998":17,"14":[24,25,51,53,57,64],"14005":17,"14006":17,"14007":17,"14008":17,"14009":17,"14011":17,"14012":17,"14015":17,"1402":24,"14023":17,"14024":17,"14033":17,"14037":17,"1404":24,"14041":17,"14059":17,"14070":17,"14081":17,"14083":17,"14086":17,"14087":17,"14089":17,"14090":17,"14092":17,"14093":17,"14094":17,"14096":17,"14100":17,"14102":17,"1412":24,"14124":17,"14125":17,"14128":17,"14137":17,"14138":17,"14141":17,"14148":17,"14153":17,"14174":17,"14183":17,"14189":17,"14207":17,"14208":17,"14211":17,"14234":17,"14238":17,"14256":17,"14257":17,"14258":17,"14260":17,"14261":17,"14263":17,"14265":17,"1427":24,"14283":17,"14285":17,"14289":17,"14293":17,"143":[17,53],"1430":54,"14305":17,"14309":17,"14310":17,"14314":17,"14317":17,"14336":17,"14343":17,"14345":17,"1435":24,"1437":24,"14371":17,"14374":17,"14377":17,"14378":17,"14379":17,"14382":17,"14384":17,"14386":17,"14392":17,"14395":17,"14406":17,"14408":17,"14425":17,"14439":17,"14446":17,"14452":17,"14457":17,"14458":17,"14486":17,"14493":17,"145":[14,53],"14505":17,"14513":17,"14525":17,"14527":17,"14528":17,"14529":17,"14539":17,"14548":17,"14558":17,"14563":17,"14571":17,"14573":17,"14574":17,"1459":24,"14596":17,"146":14,"1460":24,"14601":17,"14606":17,"14609":17,"14610":17,"14644":17,"14650":17,"14651":17,"14652":17,"14657":17,"14660":17,"14662":17,"14664":17,"14666":17,"14668":17,"14669":17,"14670":17,"14671":17,"14672":17,"14673":17,"14678":17,"14679":17,"14683":17,"14685":17,"14687":17,"14693":17,"14695":17,"14696":17,"14697":17,"14699":17,"14705":17,"14708":17,"14713":17,"14718":17,"14722":17,"14731":17,"14732":17,"14734":17,"14736":17,"14750":17,"14758":17,"14780":17,"14787":17,"14801":17,"14802":17,"14809":17,"14813":17,"14819":17,"14841":17,"14843":17,"14844":17,"14848":17,"14863":17,"14872":17,"14874":17,"14879":17,"14892":17,"14899":17,"14901":17,"14907":17,"14928":17,"14930":17,"14938":17,"14940":17,"14957":17,"14959":17,"14963":17,"14967":17,"14975":17,"14984":17,"14986":17,"14989":17,"14996":17,"15":[2,13,25,52,53,57,59,66],"150":[17,55],"15015":17,"15020":17,"15043":17,"15046":17,"15056":17,"15059":17,"15070":17,"15072":17,"15075":17,"15076":17,"15078":17,"15081":17,"15085":17,"15098":17,"15099":17,"151":77,"15121":17,"15122":17,"15139":17,"15171":17,"15193":17,"15194":17,"152":77,"15204":17,"15206":17,"15214":17,"15215":17,"15220":17,"15221":17,"15244":17,"15245":17,"15250":17,"15256":17,"15268":17,"15272":17,"15274":17,"15277":17,"15279":17,"15280":17,"15289":17,"15291":17,"15294":17,"153":53,"15300":17,"15314":17,"15322":17,"15333":17,"15334":17,"15335":17,"15338":17,"15340":17,"15347":17,"15355":17,"15366":17,"15378":17,"15382":17,"15385":17,"15388":17,"15397":17,"15403":17,"15410":17,"15411":17,"15412":17,"15420":17,"15424":17,"15426":17,"15427":17,"15432":17,"15434":17,"15442":17,"15446":17,"15448":17,"15451":17,"15483":17,"15494":17,"15496":17,"15497":17,"15498":17,"155":14,"15511":17,"15526":17,"15527":17,"15531":17,"15532":17,"15537":17,"15554":17,"15559":17,"15560":17,"15567":17,"15568":17,"15575":17,"15577":17,"15578":17,"15581":17,"15596":17,"15597":17,"15599":17,"15600":17,"15606":17,"15612":17,"15619":17,"15620":17,"15621":17,"15628":17,"15633":17,"15634":17,"15637":17,"15644":17,"15650":17,"15652":17,"15653":17,"15657":17,"15662":17,"15668":17,"15669":17,"15675":17,"15683":17,"15690":17,"15693":17,"157":53,"15714":17,"15719":17,"15725":17,"15728":17,"15733":17,"15741":17,"15745":17,"15752":17,"15754":17,"15760":17,"15778":17,"15788":17,"15789":17,"15799":17,"15802":17,"15814":17,"15838":17,"15839":17,"15843":17,"15853":17,"15861":17,"15864":17,"15866":17,"15867":17,"15873":17,"15882":17,"15884":17,"15886":17,"15888":17,"15893":17,"15903":17,"15912":17,"15921":17,"15933":17,"15938":17,"15939":17,"15945":17,"15947":17,"15964":17,"15965":17,"15967":17,"15983":77,"15984":17,"15986":17,"15996":17,"15e":17,"16":[2,25,53,54,57,59,60,71],"160":14,"16004":17,"16005":17,"16007":17,"16015":17,"16023":17,"16026":17,"16030":17,"16040":17,"16046":17,"16062":17,"16063":17,"16066":17,"16069":52,"16070":17,"16096":17,"161":14,"16101":17,"16106":17,"16118":17,"16126":17,"16135":17,"16141":17,"16142":[17,52],"16158":17,"16168":17,"16179":17,"16184":17,"16186":17,"162":[14,53],"16203":17,"16217":17,"16224":17,"16230":17,"16258":17,"16262":17,"16268":17,"16282":17,"16287":17,"16288":17,"16289":17,"16293":17,"163":[53,77],"16302":17,"16308":17,"16322":17,"16323":17,"16329":17,"16340":17,"16355":17,"16375":17,"16395":17,"16407":17,"16409":17,"16411":17,"16413":17,"16414":17,"16415":17,"16418":17,"16429":17,"16434":17,"16436":17,"16438":17,"16440":17,"16466":17,"16472":17,"16479":17,"16485":17,"16489":17,"16498":17,"165":14,"16512":17,"16519":17,"16531":17,"16535":17,"16536":17,"16537":17,"16538":17,"16540":17,"16547":17,"16552":17,"16556":17,"16571":17,"16588":17,"16602":17,"16605":17,"16632":17,"16645":17,"16651":17,"16655":17,"16659":17,"16670":17,"16677":17,"16686":17,"16690":17,"16725":17,"16731":17,"16738":17,"16740":17,"16743":17,"16752":17,"16756":17,"16757":17,"16764":17,"16765":17,"16768":17,"16785":17,"16788":17,"16796":17,"168":14,"16817":17,"16829":17,"16831":17,"16837":17,"16842":17,"16843":17,"16845":17,"16850":17,"16859":17,"16874":17,"16890":17,"16892":17,"169":[14,17],"16902":17,"16903":17,"16904":17,"16906":17,"16909":17,"16910":17,"16911":17,"16914":17,"16915":17,"16918":17,"16920":17,"16925":17,"16926":17,"16929":17,"16931":17,"16937":17,"16945":17,"16947":17,"16957":17,"16958":17,"16959":17,"16960":17,"16981":17,"16988":17,"16989":17,"16991":17,"16992":17,"16994":17,"16996":17,"16997":17,"16999":17,"16th":[24,77],"17":[24,25,27,53,57],"170":14,"17008":17,"17010":17,"17013":17,"17015":17,"17021":17,"17022":17,"17023":17,"17027":17,"17035":17,"17036":17,"17038":17,"17042":17,"17045":17,"17050":17,"17069":17,"17071":17,"17073":17,"17079":17,"17082":17,"17090":17,"17094":17,"17108":17,"17110":17,"17113":17,"17114":17,"17115":17,"17116":17,"17117":17,"17118":17,"17123":17,"17137":17,"17138":17,"17172":17,"17173":17,"17174":17,"172":54,"17206":17,"17217":17,"17221":17,"17232":17,"17258":17,"17270":17,"17274":17,"17281":17,"17285":17,"17295":17,"173":[2,14],"17303":17,"17304":17,"17305":17,"17316":17,"17318":17,"17321":17,"17322":17,"17324":17,"17333":17,"17344":17,"17347":17,"17352":17,"17359":17,"17364":17,"17371":17,"17382":17,"17392":17,"17394":17,"174":14,"17403":17,"17411":17,"17417":17,"17427":17,"17430":17,"17451":17,"17452":17,"17467":17,"17468":17,"17475":17,"17477":17,"17478":17,"17484":17,"17488":17,"17489":17,"17491":17,"17495":17,"175":77,"17503":17,"17508":17,"17534":17,"17541":17,"17544":17,"17560":17,"17564":17,"17575":17,"17576":17,"17585":17,"17591":17,"17594":17,"17597":17,"17646":17,"17660":77,"17667":17,"17669":17,"17670":17,"17697":17,"17702":17,"17704":17,"17716":17,"17718":17,"17721":17,"17732":17,"17733":17,"17734":17,"17743":17,"17744":17,"17745":17,"17747":17,"17754":17,"17760":17,"17772":17,"17774":17,"17777":17,"17782":17,"17787":17,"17788":17,"17789":17,"17794":17,"17795":17,"17796":17,"17801":17,"17805":17,"17808":17,"17817":17,"17832":17,"17836":17,"17841":17,"17844":17,"17845":17,"17854":17,"17856":17,"17857":17,"17860":17,"17861":17,"17871":17,"17872":17,"17887":17,"17889":17,"17891":17,"17892":17,"17894":17,"17897":17,"17902":17,"17927":17,"17934":17,"17935":17,"17936":17,"17946":17,"17959":17,"17963":17,"17964":17,"17984":17,"17985":17,"17986":17,"17987":17,"17988":17,"17991":17,"17993":17,"17998":17,"18":[4,13,25,57,58,59,60,64],"18004":17,"18005":17,"18006":17,"18008":17,"18014":17,"18017":17,"18022":17,"18025":17,"18026":17,"1803":17,"18032":17,"18038":17,"18059":17,"18067":17,"18068":17,"18076":17,"18077":17,"18082":17,"18089":17,"18094":17,"18095":17,"18096":17,"18102":17,"18104":17,"18106":17,"18139":17,"18151":17,"18152":17,"18157":17,"18158":17,"18159":17,"18163":17,"18164":17,"18165":17,"18172":17,"18176":17,"18183":17,"18190":17,"18193":17,"18194":17,"18195":17,"18197":17,"18209":17,"18212":17,"18223":17,"18224":17,"18230":17,"18239":17,"18243":17,"18248":17,"18254":17,"18270":17,"18273":17,"18281":17,"18292":17,"18293":17,"18298":17,"18299":17,"18311":17,"18325":17,"18327":17,"18331":17,"18342":17,"18351":17,"18359":17,"18370":17,"18374":17,"18380":17,"18392":17,"18393":17,"18395":17,"184":77,"18411":17,"18424":17,"18432":17,"18434":17,"18442":17,"18444":17,"18445":17,"18447":17,"18448":17,"18449":17,"18458":17,"18463":17,"1850":53,"18500":17,"18501":17,"18503":17,"18507":17,"18516":17,"18523":17,"18524":17,"18527":17,"18536":17,"18537":17,"18538":17,"18539":17,"18544":17,"18548":17,"18550":17,"18551":17,"18556":17,"18558":17,"18560":17,"18563":17,"18564":17,"18565":17,"18576":17,"18577":17,"18580":17,"18588":17,"1859":17,"18590":17,"18591":17,"18594":17,"18596":17,"18599":17,"186":17,"18601":17,"18604":17,"18616":17,"18618":17,"18628":17,"18630":17,"18635":17,"18636":17,"18640":17,"18641":17,"18649":17,"18656":17,"18657":17,"18662":17,"18668":17,"18670":17,"18682":17,"18690":17,"18705":17,"18706":17,"18707":17,"18713":17,"18716":17,"18717":17,"18725":17,"18729":17,"18741":17,"18743":17,"18754":17,"18757":17,"18764":17,"18765":17,"18766":17,"18769":17,"18770":17,"18771":17,"18772":17,"18785":17,"18818":17,"18834":17,"18852":17,"18863":17,"18867":17,"18873":17,"18880":17,"18887":17,"18895":17,"18906":17,"18909":17,"18910":17,"18914":17,"18915":17,"18920":17,"18921":17,"18929":17,"18936":17,"18940":17,"18942":17,"18945":17,"18947":17,"18951":17,"18958":17,"18960":17,"18973":17,"18983":17,"18988":17,"18989":17,"18th":24,"19":[24,25,41,57,77],"19006":17,"19016":17,"19017":17,"19027":17,"19032":17,"19040":17,"19049":17,"19060":17,"19069":17,"19082":17,"19088":17,"19092":17,"19096":17,"19099":17,"19100":17,"19115":17,"1912":17,"19129":17,"19136":17,"19137":17,"19138":17,"19141":17,"19144":17,"19149":17,"19152":17,"19153":17,"19164":17,"19166":17,"19179":17,"19188":17,"19197":17,"192":53,"19201":17,"19204":17,"19213":17,"19216":17,"19229":17,"19250":17,"19254":17,"19257":17,"19262":17,"19263":17,"19269":17,"19277":17,"19295":17,"19296":17,"19300":17,"19310":17,"19327":17,"19329":17,"19360":17,"19361":17,"19362":17,"19370":17,"19378":17,"19382":17,"19383":17,"19390":17,"19417":17,"19428":17,"19436":17,"19473":17,"19479":17,"19483":17,"19501":17,"19515":17,"19517":17,"19519":17,"19528":17,"19541":17,"1955":77,"1956":17,"19575":17,"1958":77,"19589":17,"19590":17,"1960":24,"19614":17,"19621":17,"19624":17,"19630":17,"19640":17,"1965":24,"19653":17,"19655":17,"19658":17,"19661":17,"19668":17,"19671":17,"19673":17,"19675":17,"19678":17,"197":77,"1970":24,"19703":17,"19704":17,"1972":77,"19730":17,"19748":17,"19749":17,"19750":17,"19752":17,"19767":17,"19768":17,"19773":17,"1980":77,"1981":77,"1982":77,"1983":24,"1984":24,"1985":[24,77],"1986":[24,77],"1987":24,"1988":[24,77],"1989":[24,77],"1990":[24,77],"1991":[24,77],"1992":[24,77],"1993":[24,77],"1994":[24,77],"1995":[24,77],"1996":24,"1997":77,"1998":[24,77],"1999":24,"19th":24,"1_000_000":29,"1a":54,"1b":54,"1beta":25,"1cvaclvffya5r":51,"1gamma":25,"1p_1":34,"1st":[24,27,34,46,57,59,64,71,72],"2":[0,1,2,3,4,5,6,7,8,9,10,11,12,13,14,15,16,18,19,20,21,22,23,25,26,27,28,29,30,31,32,33,34,35,36,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,68,69,70,71,72,73,74,75,76,77],"20":[2,25,46,57,67,77],"200":[17,52,71],"2000":[17,77],"2001":[24,77],"2002":[24,77],"2003":24,"2004":17,"2005":77,"2006":17,"2007":77,"2008":[17,77],"2010":17,"2011":[17,77],"2013":77,"2015":[17,24],"2016":17,"2017":17,"2018":17,"2019":[17,77],"2020":17,"2021":[17,77],"2022":17,"2023":17,"2024":17,"2034574":77,"2034798":77,"2051":77,"207":77,"208":53,"2080":17,"2089":17,"209":77,"20x":17,"21":54,"2100":17,"2104":17,"212":77,"214f":17,"216":77,"2168":17,"2188":17,"2190":17,"21ff":17,"22":[10,12,54,57,71],"2200":17,"2236":17,"228":77,"22ff":17,"22nd":24,"2300":17,"231":53,"2336":17,"235":77,"2357":17,"236u":53,"237":77,"2372":8,"239":53,"23ff":17,"24":[11,17,44,53,77],"240":51,"246":77,"2489":17,"24th":24,"25":[11,44,64],"2500":17,"252":77,"25379":77,"255":[27,51],"2555":17,"256":2,"256mb":51,"25th":24,"26":[53,54,77],"2600":17,"262":17,"2642":51,"2680":17,"2693":17,"26ff":17,"27":[53,54],"2700":77,"28":[54,77],"2828":17,"285":17,"28756":54,"2884":17,"28x":11,"29":60,"2900":17,"297f":17,"2_5":77,"2a00":17,"2aff":17,"2ap":17,"2nd":[24,34,41,46,57,67,72,77],"2x":[5,11],"2y":5,"3":[0,1,2,3,4,5,6,7,8,9,10,11,12,13,14,15,16,18,19,20,21,22,23,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,72,73,74,75,76,77],"30":[11,17,24,27,71],"300":[17,24],"3051":17,"31":[17,27],"3115":17,"3132":17,"3166":17,"31st":24,"32":[2,17,36,51,53,66],"3209":17,"3219":17,"328":77,"3282":17,"3290316":77,"32mword":51,"33":53,"337720":53,"337876":53,"34":[11,53,71,77],"3415":17,"3434341":77,"345":77,"3479":17,"3488":17,"35":[17,27,53],"3527":17,"3556":17,"356":17,"357":77,"36":57,"3613":17,"362":77,"3632":17,"3659":17,"37":[53,77],"3763":77,"377":77,"3826":17,"384":17,"387":52,"3886":17,"3889":17,"3890":17,"39":[17,53,71],"3941":17,"3943":17,"394648":53,"394700":53,"395448":53,"39634":77,"3977":17,"3989":17,"3994":17,"3em":[26,31,34,35,38],"4":[0,1,2,3,4,5,6,7,8,9,10,11,12,13,14,15,16,18,19,20,21,22,23,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],"40":[14,17,27,41,71],"400":17,"4007":17,"4013":17,"4041":14,"4045":14,"4056":17,"4069":17,"4095":17,"4097":17,"41":[17,51,53,57],"4105":17,"4123":17,"4129":17,"414":17,"4156":17,"4167":17,"421":17,"4250":17,"43":[17,53,54],"4306":17,"4369":17,"4373":17,"4398":17,"44":17,"4413":17,"4415":17,"4416":17,"4436":17,"4450":17,"4476":64,"4495":17,"45":[17,77],"450":17,"4502":77,"4503":17,"4504":17,"4506":17,"4511":17,"45184":53,"4519":17,"4522":17,"4529":17,"4530":17,"4533":17,"4537":17,"4540":17,"4542":17,"4544":17,"4547":17,"4548":17,"4555":17,"4574":17,"4580":17,"4582":17,"4588":17,"4591":17,"4593":17,"4596":17,"46":[11,77],"4603":17,"4606":17,"4607":17,"4608":17,"4614":17,"4623":17,"4627":17,"4630":17,"4632":17,"4638":17,"4644":17,"4673":17,"4677":17,"4683":17,"4690":17,"4696":17,"47":53,"470":17,"4709":17,"4712":17,"4718":17,"4720":17,"4721":17,"4725":17,"4738":17,"4741":17,"4747":17,"4752":17,"4754":17,"4762":17,"4769":17,"4776":64,"4777":17,"4780":17,"48":[17,51],"4818":17,"4822":17,"4823":17,"4824":17,"4832":17,"4841":17,"4844":17,"4851":17,"4858":17,"4863":17,"4871":17,"4876":17,"4880":17,"4881":17,"4882":17,"4887":17,"4890":17,"49":77,"4911":17,"4912":17,"4925":17,"4947":17,"4969":17,"4970":17,"498":66,"4994":17,"4beta":25,"4beta2":25,"4th":[24,41,44,77],"5":[0,1,2,3,4,5,6,7,8,9,10,11,12,13,14,15,16,18,19,20,21,22,23,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],"50":[17,27,41,42,44,53,57,59,71,77],"500":17,"5001":17,"5007":17,"5008":17,"5019":17,"5026":17,"5030":17,"5043":17,"5062":17,"5065":17,"5077":17,"5095":17,"5097":17,"51":17,"5102":17,"512":2,"5123":17,"5127":17,"5132":17,"5150":17,"5155":17,"5159":17,"5163":17,"5173":17,"52":53,"5205":17,"522":17,"5222":17,"5223":17,"5233":17,"52335":77,"5239":17,"5244":17,"5248":17,"5255":17,"5275":17,"5300":17,"5304":17,"5308":17,"5315":17,"532":64,"532u":64,"5336":17,"5351":17,"5360":17,"5365":17,"5369":17,"5377":17,"5380":17,"5384":17,"5390":17,"5394":17,"54":17,"540":77,"5414":17,"5417":17,"5420":17,"5435":17,"5439":17,"5445":17,"5449":17,"5475":17,"5476":17,"5481":17,"5482":17,"5486":17,"5487":17,"55":17,"5501":17,"5507":17,"5520":17,"5521":17,"5522":17,"5523":17,"5524":17,"5526":17,"5535":17,"5546":17,"5548":17,"5550":17,"5553":17,"5568":17,"5574":17,"5577":17,"5578":17,"5589":17,"5597":17,"5598":17,"5607":17,"5618":17,"5619":17,"5620":17,"5641":17,"5648":17,"5651":17,"5671":17,"56772":53,"56980":53,"57":[17,54],"5702":17,"5706":17,"5726":17,"5730":17,"5752":17,"5764":17,"5777":17,"581478":77,"581501":77,"582153":77,"582176":77,"59":[17,57],"592":53,"5941":17,"5_13":77,"5beta1":25,"5beta2":25,"5beta3":25,"5d4558edf8f5c2c548a3d96c17820169":17,"5pl1":25,"5pl2":25,"5pl3":25,"6":[2,9,25,29,35,53,54,55,57,58,71,74,77],"60":[27,53],"6042":17,"6092":17,"61":[17,53],"6109":17,"6134":17,"6261":17,"6278":17,"63":[5,17,29,36,71],"6332":17,"64":[2,36,51,66],"642":77,"6459":17,"650":[17,24,54],"66":[53,77],"664":77,"6677":17,"6705":17,"6714":17,"6720":17,"6785":17,"68":[46,53],"6857":17,"69":[53,71],"6914":17,"6976":17,"6beta1":25,"6f62bda":17,"6th":24,"7":[2,11,25,54,57,64,71,74,75,77],"70":[17,27,36,42,57,71,72],"7015":17,"7017":17,"7086":77,"709":77,"7093":17,"71":46,"7135":17,"72":46,"720":77,"7221":17,"7253":17,"7309":17,"7333":17,"7348":17,"7385":17,"7393":17,"74":53,"7443":17,"7462":17,"75":[17,27,71],"7522":17,"75277":77,"75285":77,"754":[17,36],"757":17,"7615":17,"7632":17,"7634":17,"7674":17,"7675":17,"7695":17,"7697":17,"7698":17,"772":17,"7723":17,"7725":17,"7730":17,"7766":17,"7769":17,"7791":17,"78":59,"7812":17,"7825":17,"7886":17,"7894":17,"7902":17,"7911":17,"7913":17,"7916":17,"7979":17,"7982":17,"7998":77,"7edelahay":77,"7x":11,"8":[2,4,13,24,25,27,30,35,41,51,52,53,54,57,58,59,60,64,66,71,75],"80":[27,71],"8032":17,"8062":17,"8080":17,"8094":17,"8161":17,"8171":17,"8176":77,"82":77,"8215":17,"8217":17,"8252":17,"8276":17,"836":53,"8365":17,"8388607":17,"8388851":17,"84":77,"8402":17,"8419":17,"8451":17,"8457":17,"8459":17,"8481":54,"8488":17,"85":[27,53,71,77],"8540":17,"8555":17,"8560":17,"8638":17,"8642":17,"8649":17,"8667":17,"8669":17,"87":[24,53],"872":17,"8739":17,"874":17,"8764":17,"8779":17,"8791":17,"88":[24,53,77],"8808":17,"8815":17,"8817":17,"8819":17,"8820":17,"8829":17,"8850":17,"8855":17,"8859":75,"8870":17,"8898":17,"89":[53,54,77],"8905":17,"8920":17,"8945":17,"8965":17,"8987":17,"8989":17,"8991":17,"8_62":77,"8th":24,"9":[2,24,25,29,30,35,53,54,57,64,71,74,77],"9000":17,"9001":17,"9013":17,"9058":17,"9078":17,"9086":17,"9095":17,"9098":17,"91":[7,60,77],"9114":17,"9117":17,"9133":17,"9142":17,"9146":66,"9148":17,"9160":17,"9162":17,"92":[54,77],"9214":17,"9270":17,"9274":17,"9279":17,"9288":17,"9294":17,"93":[10,53],"9300":17,"9306":17,"9307":17,"9319":17,"9336":17,"9341":17,"9363":17,"9364":17,"9379":17,"94":77,"9403":17,"9410":17,"9425":17,"947":77,"9490":17,"95":[27,60,77],"9508":17,"9509":17,"9512":17,"9514":17,"9517":17,"9519":17,"9521":17,"9524":17,"9530":17,"9532":17,"9555":17,"9569":17,"96":53,"9602":17,"9608":17,"9637":17,"9651":17,"9668":17,"9670":17,"9681":17,"9682":17,"9696":17,"97":[53,77],"9705":17,"9711":17,"9716":17,"9725":17,"9741":17,"9743":17,"9767":17,"9772":17,"978":77,"9803":17,"9811":17,"9816":17,"9825":17,"9829":17,"9840":17,"9844":17,"9848":17,"9851":17,"9854":17,"9856":17,"9867":17,"9872":17,"9874":17,"9876":17,"9883":17,"9884":17,"9885":17,"99":[17,27,71],"9906":17,"9918":17,"9939":17,"996":77,"9964":17,"9971":17,"9979":17,"9984":17,"9995":17,"9996":17,"9_":71,"9_26":77,"9_47":77,"9e":77,"9th":77,"\u00e0":[17,24,55],"\u00e8":77,"\u00e9":77,"\u00e9cole":24,"\u00e9lie":17,"\u00eb":77,"\u015ferb\u0103nu\u0163\u0103":17,"\u03b1":[3,14,25,54,55,57],"\u03b2":[17,25,26,57],"\u03b2\u03b4\u03b9":11,"\u03b2\u03b4\u03b9\u03b6":[0,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],"\u03b2\u03b4\u03b9\u03b6\u03b7":[14,26,31,34,35],"\u03b2\u03b9":[17,41,57,64],"\u03b2\u03b9\u03b6":64,"\u03b2v":55,"\u03b3":[14,26,31,34,35,38,55],"\u03b3_":[26,34],"\u03b3_1":[26,34],"\u03b3_2":26,"\u03b3_c":[26,34,35,38],"\u03b3_i":[26,34,35,38],"\u03b3_n":34,"\u03b3_p":[26,34,35],"\u03b4":[25,26,37,41,57,64,67],"\u03b6":[25,26,57],"\u03b7":[12,17,25,30],"\u03b7\u03b6":57,"\u03b9":[25,26,34,41,55,64],"\u03bb":[17,24,26,31,34,38,52,54,57,66,77],"\u03bbp":34,"\u03bbprolog":63,"\u03bbs":52,"\u03bbx":[26,31,34],"\u03bbz":34,"\u03c0":52,"\u03c1":57,"\u03c3":[35,67],"\u03c6":[17,64,71],"\u03c9":77,"\u2115":39,"a\u2081":4,"a\u2096":4,"abstract":[2,4,5,11,13,14,17,24,25,26,27,28,29,34,35,38,42,44,54,55,58,59,64,67,71],"andr\u00e8":17,"ar\u00eda":17,"arma\u00ebl":17,"bj\u00f6rn":17,"boolean":[2,5,9,11,13,14,17,24,25,27,29,34,37,39,40,42,55,59,60,62,64,67,71],"break":[10,12,17,28,29,30,52,57,59,64,66,71,73,74],"byte":[17,24,25,27,51,59,66,71],"c\u00e9dric":17,"case":[0,1,2,3,4,6,7,8,9,10,11,12,13,14,15,16,17,18,19,20,21,22,23,25,26,27,28,29,30,31,32,33,34,35,36,37,38,39,41,42,43,44,45,46,47,48,49,50,51,53,54,55,56,59,60,61,62,63,64,65,66,68,69,70,71,72,73,74,75,76,77],"cast\u00e9ran":[17,77],"catch":[3,17,25,42,46,57],"char":[2,17,53],"chargu\u00e9raud":17,"chrz\u0105szcz":[17,24],"cl\u00e9ment":[3,17],"class":[13,17,24,25,27,28,35,39,42,44,57,59,60,62,64],"const":[26,34,37,54],"cr\u00e9gut":24,"d\u00e9mon":24,"d\u00e9monstrat":77,"d\u00e9n\u00e8":17,"default":[2,3,4,5,8,9,10,11,12,13,14,17,24,25,27,28,29,32,34,35,37,38,43,44,51,52,53,54,55,57,58,59,60,62,64,66,67,71,74,75],"do":[2,3,4,7,8,10,13,14,17,24,25,27,29,31,32,34,35,37,38,42,46,51,52,53,55,57,58,59,60,62,63,64,66,67,71,74,75],"double":57,"export":[3,5,9,11,13,17,24,27,29,35,38,51,52,54,55,59,60,71],"f\u03c9":24,"f\u2081":4,"f\u2096":4,"f\u2099":4,"filli\u00e2tr":[2,17,24,77],"final":[2,3,4,5,6,8,9,10,11,13,14,17,24,25,27,29,35,40,51,52,53,54,57,59,64,66,67,71,75],"float":[14,17,24,25,34,59,71],"formalis\u00e9":24,"fr\u00e9d\u00e9ric":[5,17,57],"fr\u00e9deric":17,"fran\u00e7oi":[17,57],"franti\u0161ek":17,"function":[2,3,5,9,10,11,12,13,14,17,24,25,26,27,31,33,35,36,37,39,42,45,46,51,52,55,57,58,59,62,64,67,71,73,77],"g\u00e1sp\u00e1r":17,"g\u00e9rard":[24,77],"g\u00f6teborg":24,"ga\u00ebtan":17,"gim\u00e9nez":[24,77],"gr\u00e9goir":[11,17],"gr\u00f6bner":[7,17],"grabovsk\u00fd":17,"gu\u00e9neau":17,"hu\u1ef3nh":17,"ident\u2081":46,"ident\u2099":46,"import":[2,3,4,5,6,7,9,11,13,17,24,25,26,27,28,29,31,32,34,35,36,38,40,42,43,44,51,52,53,54,55,57,58,59,60,62,64,66,67,71,72],"int":[2,3,17,27,36,55,71,75],"j\u00e9r\u00f4me":24,"jes\u00fa":17,"judica\u00ebl":24,"ko\u0161\u00edk":17,"l\u00e9chenet":17,"l\u00e9o":17,"l\u00f6f":[24,27,34],"laulh\u00e8r":24,"leli\u00e8vr":17,"lo\u00efc":[7,17,24],"long":[8,14,17,25,30,51,52,53,58,59,67,71],"march\u00e9":[17,24],"mat\u011bj":17,"math\u00e9matiqu":24,"mu\u00f1oz":[24,77],"new":[4,5,6,8,10,13,14,15,25,27,29,31,32,34,36,37,39,42,43,46,51,52,54,55,58,60,61,64,66,67,71,72,73,75,77],"null":[17,24,27,57],"p\u00e9drot":17,"public":[14,17,25,50,59,74],"q\u2081":17,"q\u2082":17,"r\u00e9alis":24,"r\u00e9gi":17,"rapha\u00ebl":17,"return":[0,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],"s\u00e9bastien":17,"sa\u00efbi":[4,24],"short":[8,14,17,24,25,31,35,36,38,51,53,55,57,59,64,75],"st\u00e9phane":17,"static":[17,24,25,53,71],"sup\u00e9rieur":24,"super":64,"switch":[3,8,13,14,17,24,25,51,53,66],"synth\u00e8s":24,"t\u2081":4,"t\u2098":4,"t\u2099":4,"th\u00e8se":77,"th\u00e9o":17,"th\u00e9ori":77,"th\u00e9ry":[11,17,24],"throw":[17,55],"tr\u1ea7n":17,"triangleright_\u03b2":31,"triangleright_\u03b4":[31,35],"triangleright_\u03b6":31,"triangleright_\u03b7":31,"triangleright_\u03b9":34,"true":[2,4,5,7,9,11,12,13,14,17,24,26,27,34,35,36,37,40,41,44,46,51,53,54,55,57,58,59,62,64,67,71,74],"try":[2,3,11,14,17,24,25,34,35,40,41,43,46,53,55,57,60,62,64,66,67,71],"trzci\u0144ski":17,"u\u2081":4,"u\u2098":4,"universit\u00e9":77,"v\u1d62":55,"v\u2080":55,"v\u2081":4,"v\u2099":[4,55],"var":[17,24,26,54,58],"void":17,"w\u2081":51,"w\u2099":51,"while":[2,3,4,9,10,12,13,14,17,24,25,26,27,28,29,31,32,33,34,35,36,37,40,41,42,43,44,46,51,52,53,54,55,57,58,59,60,62,63,64,66,67,71,73],"x\u1d62":55,"x\u2080":55,"x\u2081":4,"x\u2096":4,"x\u2099":[4,55],A:[3,4,5,7,9,10,11,12,13,17,24,25,26,27,28,29,30,31,32,34,36,37,38,39,40,41,42,43,44,46,50,51,52,53,54,55,57,59,60,62,63,64,66,71,72,74,75,76,77],And:[42,51,53,54,71],As:[2,3,5,6,9,10,11,13,14,17,26,28,30,34,36,37,38,41,42,43,44,46,51,52,53,54,55,57,58,59,60,66,67,71,72],At:[8,11,14,24,26,27,33,34,42,51,52,54,55,57,59,60,71,74],BE:2,Be:[17,75],But:[2,11,17,34,39,41,46,51,53,54,64,75],By:[3,4,5,11,12,13,14,17,29,34,37,44,46,51,53,54,55,57,60,64,66,67,71],For:[2,3,4,5,7,8,9,11,12,13,14,16,17,24,26,27,28,29,30,31,34,35,36,37,38,40,41,42,43,44,45,46,51,52,53,54,55,57,58,59,60,62,64,66,67,71,72,75],IF:[17,71],IS:71,If:[2,3,4,5,7,8,9,10,11,13,14,17,26,28,29,30,32,34,35,37,38,39,41,42,44,46,51,52,53,54,55,57,58,59,60,62,64,66,67,71,72,73,74,75],In:[0,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,56,57,58,59,60,61,62,63,64,65,66,67,68,69,70,71,72,73,74,75,76,77],Is:[25,66],It:[2,3,4,5,6,7,8,9,10,11,12,13,14,17,24,25,27,28,29,30,31,32,34,35,37,38,40,41,42,44,46,51,52,53,54,55,57,58,59,60,62,64,66,67,71,72,74,75],Its:[3,11,17,24,52,55,57,60,67,74],NO:57,No:[3,5,6,9,11,12,13,14,17,24,25,26,30,34,35,36,40,42,44,54,55,57,58,59,60,62,64,66,67,71,72,74],Not:[11,17,27,32,44,51,52,54,55,58,64,67,72,75,77],Of:[2,14,42,51,57],On:[3,10,12,17,24,27,30,32,37,40,44,46,51,52,53,54,57,58,64,71],One:[3,8,9,13,14,17,25,31,32,34,37,38,39,44,51,53,54,55,59,60,64,66,67,71,75],Or:[12,17,41,53,58,71],Such:[12,30,35,42,44,53,55,59,71,75],TO:2,That:[3,27,29,30,34,36,52,54,55,58,64,66],The:[2,3,4,5,6,8,9,10,12,13,14,15,17,24,25,28,29,30,31,32,33,36,37,38,39,40,41,42,43,46,52,54,55,58,59,60,62,63,64,65,66,67,72,73,74,76,77],Their:[3,17,32,34,39,55,57,59,71],Then:[2,4,5,11,14,24,26,27,29,32,34,41,42,46,51,53,54,55,57,58,59,60,64,65,66,67,71,74,75],There:[4,9,10,11,14,17,24,25,26,27,28,29,34,37,38,39,40,44,46,51,52,53,54,55,57,58,59,60,63,64,66,67,71,72,75],These:[3,11,13,14,17,24,25,27,28,29,31,32,34,36,37,38,40,52,53,54,55,57,58,60,64,66,67,71,72,73],To:[3,4,5,6,7,8,9,10,13,14,17,24,25,27,29,30,32,34,37,39,41,42,44,46,51,52,53,54,55,57,58,59,64,66,67,71,72,74,75],WITH:35,With:[3,4,13,14,17,46,53,57,58,67,71],_0:17,_1:35,_:[0,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],__arith:5,__ff:5,__varmap:5,__wit:5,__x1:5,__x2:5,_a_:57,_and_:24,_assoc:59,_b_:57,_complet:72,_coqproject:[17,25,51,52],_correct:72,_darc:51,_e:71,_emphas:75,_eqn:17,_equat:72,_f:[41,72],_foo:17,_full:17,_h:29,_hl:[0,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],_ho:29,_hyp_:57,_i:[35,71],_ind:[34,35,40,71,72],_invol:17,_involut:17,_l:[17,34],_list:71,_list_sep:71,_m:35,_morphism:3,_mybool_scop:41,_n_:57,_not_:17,_p:71,_pack:42,_r:[17,41],_rec:[2,34,35,40,71,72],_rect:[2,17,34,35,40,71,72],_scope:71,_sind:[34,35,40,71],_subproof:[17,59,66],_subterm:59,_tcc:72,_termin:72,_underscores_:17,_x:[46,57],_x_:[17,57],_xxx_:57,a0:[24,46,67],a1:[3,27,34,46,57,58,71],a2:[3,27,34,58],a3:27,a_1:[26,34,35,38],a_:34,a_i:[26,34],a_j:[34,35],a_k:[34,35],a_l:26,a_left:17,a_m:34,a_n:[34,38],a_p:34,a_r:34,a_right:17,aac:17,aaron:17,ab:[17,27,57,67,71],abadi:77,abandon:17,abbr:17,abbrevi:[4,5,13,14,17,24,25,27,32,35,38,59,74],abc:71,abdullah:17,abel:77,abezoutn:57,abhishek:17,abidin:77,abil:[2,3,11,12,13,17,30,52],abl:[3,8,11,13,14,17,24,25,34,42,44,46,51,53,55,57,58,59,61,62,67],abort:[3,11,17,34,42,44,54,55,57,64,66,67],about:[2,3,5,11,13,14,15,17,24,25,29,30,34,37,39,41,51,52,53,54,55,57,58,59,60,62,64,66,67,72],abov:[2,3,5,11,13,14,17,24,28,30,34,37,38,42,44,51,52,53,54,55,57,58,59,64,66,71,72,75],abr:24,abridg:57,abruptli:52,absenc:[9,17,71],absent:[37,59],absolut:[17,24,35,51,53,55,71],absurd:[5,27,34,51,58],absurd_hyp:17,absurd_set:27,abus:[2,55],ac19:[12,77],academ:77,acc:[17,27,34,35],acc_in:34,acc_ind:34,acc_intro:27,acc_inv:27,acc_it:17,acc_iter2:17,acc_rec:34,acc_rect:[17,27,34],acc_simul:17,acc_sind:34,acceler:[17,52],accept:[2,3,13,17,24,28,29,30,32,34,40,44,45,46,51,52,53,54,55,57,58,60,64,66,71,72],access:[2,5,14,17,24,25,27,28,32,33,34,35,36,38,44,51,52,53,55,57,59,71],accessopaqu:17,accident:[17,57],accommod:[24,57],accompani:17,accomplish:[14,57],accord:[2,11,17,26,34,35,41,51,53,55,57,59,60,64,71],accordingli:[8,17,40],account:[5,9,13,14,17,24,26,34,37,41,44,54,57,60,67,71],accumul:54,accur:[17,52,53,57,71],accustom:57,acdsimpl:11,achiev:[7,11,13,17,24,54,57,71],achil:54,ack0:60,ack1:60,ack2:60,ack:[59,60],ackermann:59,ackm:59,acknowledg:25,acm:77,aco:17,across:[17,52,54,55,57,59,73],act:[9,17,37,46,52,54,55,67],actic:77,action:[17,24,52,53,57,60],activ:[8,9,14,17,24,25,29,32,35,37,42,43,44,46,52,53,54,59,60,64,66,71],actual:[2,3,5,8,11,14,17,24,34,37,42,43,44,46,54,55,57,60,64,67,71,72],acycl:[24,39],aczel:24,ad:[2,4,9,13,14,17,24,25,27,29,34,37,42,44,51,53,54,55,57,58,59,60,62,64,66,67,71,73,75,77],adam:17,adapt:[3,7,17,24,51,57,63],add1:[55,64],add:[3,4,5,8,9,10,11,13,14,17,24,25,27,29,31,32,34,37,41,42,44,46,51,53,54,55,57,58,59,60,62,64,66,67,71,73,75],add_0_l:17,add_assoc:[17,59],add_bottom:[17,71],add_carri:17,add_carry_div2:59,add_comm:[3,17,59,64],add_instance_attempt:42,add_last:57,add_mul:57,add_shuffle0:59,add_shuffle1:59,add_shuffle2:59,add_shuffle3:59,add_succ_comm:59,add_top:[17,71],add_transpose_neqkei:17,add_un_double_moins_un_xo:17,add_zifi:5,addit:[3,4,5,8,9,13,17,24,25,27,29,31,34,35,39,51,52,53,54,55,58,59,62,64,65,66,67,71,72,73],addition:[9,13,14,17,34,46,53,54,58,59,64,66],addn0:57,addn:57,addnc:57,addnca:57,addpath:[17,24],addr:17,addrecpath:[17,24],address:[17,52],addsn:57,addsnn:57,addx:57,adhoc:[17,37],adjac:57,adjoin:17,adjoint:17,adjointif:17,adjust:[14,17,38,71],admiss:[30,38],admit:[8,9,13,17,30,32,37,42,46,51,52,57,66],admitaxiom:17,adopt:[17,57,73,75],adrian:17,advanc:[5,17,25,33,34,42,53,54,58,64,71,74],advantag:[8,17,24,46,51,53,57,62,64,67],advertis:17,advic:[15,17],advis:[11,17,24,25,28,29,30,54,60],aeq:3,aesthet:54,affect:[12,17,24,29,34,41,44,46,53,54,55,57,59,60,64,66,71],affeldt:17,aforement:[9,51],aft:75,after:[2,4,5,7,9,11,13,17,24,29,32,34,35,38,41,42,46,51,52,53,54,55,57,58,59,60,62,64,66,67,71,72],afterward:[9,17,41,44,52,57,60,66,67],again:[3,13,17,24,34,42,52,53,55,57,60,64,66,71],against:[10,13,17,44,54,57,58,59,60,62],agda:30,aggress:57,ago:17,ahead:[17,54],aid:24,aim:66,aka:[17,72],akin:[17,30,55],akira:17,al:[3,57],al_unit:54,ala:53,alban:17,albeit:17,aleksandar:77,alessandro:77,alexand:17,alexandr:17,alexei:17,algebra:[7,14,17,24,39,42,54,55,64,77],algorithm:[3,7,9,11,13,17,24,25,41,51,54,57,59,62,66,77],algorithmica:77,ali:17,alia:[2,17,24,29,35,46,55,58,60],alias1:35,alias2:35,alias:[2,17,24,25,29,35,55],alias_definit:[55,58],align:[10,59,71],all:[2,3,4,5,7,8,9,10,11,12,13,14,17,24,26,27,28,29,30,31,34,35,36,37,38,39,40,41,42,44,46,51,52,53,54,55,57,58,59,60,62,64,66,67,71,72,73],all_eq:12,all_iff_morph:3,all_nul:57,all_sig2_cond:17,allai:17,alldfil:53,allevi:67,alloc:[17,51],allow:[2,3,4,5,7,8,9,10,11,12,13,14,17,24,25,26,27,28,29,30,31,32,34,37,38,40,42,44,46,51,52,53,54,55,57,58,59,60,62,63,64,66,67,71,72],allt:[17,24],alltact:52,almost:[3,17,57,67,75],alon:[17,24,34,67],along:[8,17,24,34,53,57,58,66,74],alongsid:17,alpha:[17,31,54,55],alpha_p:5,alphabet:[17,60],alreadi:[2,4,13,17,24,27,28,32,37,41,42,44,51,52,53,54,55,57,58,59,60,66,67,71,73],alright:2,also:[2,3,4,5,6,7,8,9,10,11,12,13,14,17,24,25,26,27,28,29,30,31,32,34,35,37,38,39,40,41,42,43,44,46,51,52,53,54,55,57,58,59,60,62,63,64,66,67,71,72,73,74,75,77],alt:[17,52],alter:[17,35,75],altern:[7,8,9,11,13,17,24,25,29,30,35,40,43,44,46,52,53,55,57,59,62,64,65,66,71,75,77],although:[3,5,9,17,35,37,53,55,57,58,60,64,66],alvarado:24,alwai:[2,3,4,6,9,10,11,12,13,14,17,24,26,34,35,37,41,42,44,51,52,53,54,55,57,58,60,66,67,71,74,75],am:55,ambient:55,ambigu:[4,17,25,46,53,57,59,60,66,71],ambiti:24,ambrois:17,amen:67,amend:42,amin:17,aminev:17,amokran:[4,24],among:[7,13,17,24,25,26,34,44,53,54,55,57,64],amorim:17,amount:[3,5,8,14,17,27,51,54,58],an:[2,3,4,5,6,7,8,9,10,11,12,13,14,17,24,25,26,27,28,29,30,31,32,34,36,37,38,39,40,41,42,43,44,46,51,52,53,54,55,58,60,62,63,64,66,71,72,74,75,77],ana:17,analog:[3,17,34,54,57,58,66],analogu:57,analys:13,analysi:[17,24,25,30,34,37,40,46,57,58,72,77],analyz:[17,27,40,57,67],anand:17,ancestor:[24,53],andE:57,and_assoc:59,and_darc:51,and_rect2:27,andb:[2,13,17,27,62],andb_comm:59,andb_negb_l:17,andb_prop:59,andb_true_intro:59,andbc:57,andp:57,andpp:17,andr:17,andrea:[17,77],andrej:17,andrew:[17,77],anew:57,angl:24,anguag:77,ani:[2,3,4,5,6,7,8,9,10,11,12,13,14,17,24,26,28,29,30,31,32,34,35,37,38,39,41,42,43,44,46,51,52,53,54,55,57,58,59,60,62,64,66,67,71,75],annoi:57,annot:[3,9,14,17,24,25,27,34,41,42,45,51,53,55,57,66],anomali:[10,17,24,59],anonym:[14,17,24,25,44,54,66],anoth:[3,4,9,11,13,14,17,24,27,31,32,34,35,40,42,43,44,46,51,52,53,54,55,57,58,59,62,63,64,66,67,71],anr:17,ansi:51,answer:[11,46,53],antialias:52,antinomi:24,antipoli:[17,24],antiquot:[17,25],antisymmetr:17,anton:17,antonia:72,antonio:17,anymor:[9,17,55,59],anyth:[2,13,17,35,44,46,51,55,57,58,64,75],anything_ind:2,anything_rec:2,anything_rect:2,anything_sind:2,anytim:54,anywai:57,anywher:[43,58,75],ap:[4,11],apart:[9,13,31,35,55],api:[8,17,25,59,63],app:[17,26,27,34,35,55,58,67],app_ass:17,app_assoc_revers:17,app_eq_app:17,app_eq_con:17,app_inj_pivot:17,app_inj_tail_iff:17,app_inv_head_iff:17,app_inv_tail_iff:17,app_length:17,app_nil_end:17,app_nth2_plu:17,app_rlist:17,appar:[14,17,51,54,57],apparatu:9,appart:51,appcontext:17,appdata:52,appeal:27,appear:[2,6,9,10,11,13,14,17,24,28,29,31,34,35,37,38,39,41,43,44,46,51,52,53,54,55,57,58,59,60,64,66,67,71,74,75],appel:17,append:[3,17,29,35,43,53,54,66,75],append_const:17,append_inj:17,appendix:17,appli:[2,3,4,5,9,10,11,13,14,17,24,25,26,27,28,29,30,31,32,34,35,36,37,38,40,41,42,44,46,51,53,54,55,59,60,62,66,71,72,75],applic:[3,5,10,11,13,14,17,24,25,26,29,30,35,36,37,41,46,52,55,57,59,60,64,66,67,71,72,77],apply_id:71,apply_mor:3,approach:[24,27,52,53,55,57,58,67,75],appropri:[4,13,14,17,29,53,55,57,59,62,64,66,67,75],approxim:[5,12,14,17,60],apr:17,april:[17,77],ar:[2,3,4,5,6,7,8,9,10,11,12,13,14,16,17,24,25,26,27,28,29,30,31,32,33,34,35,36,37,38,39,40,41,42,43,44,46,50,51,52,53,54,55,58,59,60,61,62,63,64,65,67,71,72,73,74,75],ar_unit:54,arab:29,arakaki:17,arbitrari:[2,3,5,10,11,14,17,24,31,44,46,53,57,60,62,71],arbitrarili:[17,58,71],archclean:53,architect:24,architectur:[17,24,29],archiv:[17,77],area:17,aren:[17,52,53,54,58,73,75],arg:[17,24,28,37,44,51,53,55,57,60,67],arg_spec:41,args_modifi:41,argument:[3,4,5,6,7,9,11,12,13,14,17,24,25,27,28,29,30,31,32,33,34,35,38,40,42,43,45,51,52,54,55,58,59,60,62,64,66,72,75],argument_spec:41,ari:[3,17,34],aria:17,aris:[3,9,13,17,30,67,71],arith:[3,5,9,11,17,24,27,43,53,57,58,59,60,64,72],arith_bas:[17,59],arith_prebas:17,arithmet:[17,24,25,36,44,57,60,61,71],arithr:11,ariti:[2,17,24,25,46,55],arnaud:17,around:[12,17,24,29,46,52,53,55,57,58,59,64,67,71,75],arr:[26,34],arrai:[0,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,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],array_get:36,array_set:36,array_typ:36,arrow:[3,4,14,17,52,57,60,64,67],art:[17,52],arthur:17,articl:24,articul:71,artifact:17,artifici:[17,24,67,71],as_ipat:58,as_nam:58,ascand:24,ascii:[17,52,53,71,75],ascii_as_ot:17,asciisyntax:17,ascrib:17,asf:77,asid:[34,64,66,67],asin:17,ask:[2,3,17,25,42,43,53],askra:59,aspect:[17,24,46],asr:17,ass:54,ass_app:17,assert:[2,17,24,25,26,28,34,41,54,55,57,58,62,64,66,67,71],assert_fail:[17,25],assert_succe:[17,25],assia:[11,17,42,57,77],assign:[13,17,25,27,29,43,51,52,53,54,55,58,66,71],assist:[17,24,25,33,65,75],assoc:54,associ:[2,3,11,13,14,17,24,25,26,27,28,29,31,32,34,35,36,37,38,42,44,46,51,52,53,54,55,57,58,59,60,64,66,67],assum:[2,3,5,11,13,17,26,27,28,32,34,35,36,38,39,42,44,46,51,53,54,55,57,58,59,64,66,71,75],assumpt:[4,10,17,24,25,26,32,33,34,35,36,44,51,52,53,54,58,59,60,66,67,77],assumption_token:[28,59],assur:[17,53],ast:[17,24,37],ast_closure_term:17,asterisk:75,asymc:52,asymmetr:[17,46],asymptot:[2,59],async:[8,17,52,54],asynchron:[17,25,66,76],atan_right_inv:17,atom:[4,5,8,14,17,26,60,62,67,71],atomic_tac2pat:55,attach:[14,17,29,52,59,71,74],attack:51,attempt:[8,14,17,24,41,52,54,66],attent:66,attila:17,attr:[17,29,51],attr_valu:29,attract:17,attribtu:14,attribut:[3,5,9,13,14,16,25,28,30,32,34,37,40,41,42,44,51,54,55,59,60,62,64,66,71,74],auger:17,august:[17,24],austin:24,author:[2,3,4,5,7,8,9,11,14,17,27,29,42,46,57,73,74],auto:[11,13,14,17,24,29,34,41,44,51,52,54,57,58,59,60,62,66,67,72],auto_us:60,autoappli:[13,17],autocomplet:17,autogener:17,autoinlin:[2,17],autom:[17,24,25,43,54,59,61,64,66,67,77],automat:[2,3,5,7,9,10,13,14,17,24,25,27,28,35,37,40,42,46,52,53,54,55,57,58,60,64,65,66,71,72,75,77],automath:24,automatiqu:77,automaton:[24,75],autonom:17,autorewit:17,autorewrit:[3,17,24,60],autounfold:[17,60],auxiliari:[8,17,34,53,54,57,66],avail:[2,9,11,12,13,17,24,25,27,30,35,36,37,38,40,42,46,50,51,52,53,54,55,57,58,59,60,62,63,64,65,66,71,72,74,75,76,77],avec:24,averag:24,avi:17,avl:[17,27],avoid:[6,8,11,12,13,17,24,25,29,34,37,52,54,55,57,58,59,60,64,66,67,71,74],awai:[17,54],await:52,awar:[17,51,52,55,58,59,62,66],awk:17,awkward:[24,54],ax:[26,44,67],axiom:[3,7,9,10,11,12,14,17,24,25,27,28,29,30,31,32,34,35,36,38,42,44,51,52,54,57,58,59,60,64,66,67,71,72,74],axiomat:[17,24,27,36,54,71],axiomatis:17,ayach:17,azevedo:17,b0:46,b1:[57,59],b2:[57,59],b2n:[41,59],b2n_le_1:17,b3:57,b:[2,3,4,8,9,10,11,12,13,14,17,24,25,27,28,31,34,35,37,38,40,41,42,44,46,50,51,52,53,54,55,57,59,60,62,64,66,67,71,72,77],b_1:34,b_:34,b_i:34,b_j:34,b_m:34,b_r:34,ba:17,back:[3,9,14,17,24,51,52,54,57,58,59,66,67],backchain:57,backend:24,background:[17,31,51,52,54,66],backport:17,backquot:17,backslash:51,backspac:52,backto:[17,59],backtrac:[17,25,55,59],backtrack:[11,13,17,24,25,52,58,60,67],backward:[17,25,51,52,55,57,63,66,71],bad:[2,11,12,14,17,34,59,64],baeld:17,bahmann:17,bail:8,bakel:17,balaa:72,balanc:[17,57],banner:24,bar0:55,bar81:[26,66,77],bar:[2,8,14,17,29,35,51,52,53,55,57,64,66,71,74],bare:[17,71],barenblat:17,barendregt:[24,77],barra:[11,17,24],barrett:17,barri:17,bart:17,barth:72,base0:60,base1:60,base:[3,5,10,11,12,13,14,17,24,25,29,33,35,39,42,43,44,51,52,53,54,55,57,58,60,62,63,64,66,67,71,73,74,75,77],base_includ:59,basenam:53,bash:[17,52],basi:[7,17,52,59],basic:[3,11,17,24,25,32,33,34,35,37,40,42,44,46,51,58,59,60,63,66,67,73],basicelim:[17,67],basicmatch:46,batch:[8,17,25,54,66],bati:17,battl:2,baz:[14,53],bazaux:53,bdd:2,bdenesgregoire11:[64,77],bear:10,beautifi:[17,51],becam:[17,24],becaus:[2,3,4,8,11,12,14,17,24,26,28,29,31,33,34,35,37,39,40,41,43,44,45,46,51,52,53,54,55,57,58,59,60,62,64,66,67,71,72],beck:17,becker:17,becom:[2,8,11,17,24,26,28,34,35,40,44,46,52,53,55,57,58,59,64,66,67,71],bedrock:17,been:[2,3,8,9,10,11,13,14,17,24,25,27,28,29,32,34,35,41,42,44,46,51,52,53,54,55,57,58,59,60,63,64,66,67,71,72,73,74],beep:71,befor:[2,4,5,13,14,17,28,29,32,34,37,41,42,44,51,52,53,54,55,57,58,59,60,64,66,67,71,73,74,75],beforehand:[17,51,55],begin:[0,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],beginn:[17,25],behalf:17,behav:[3,11,17,24,28,29,31,34,35,43,53,54,55,57,58,60,62,64,67,71],behavior:[2,3,4,11,13,14,17,24,29,30,32,34,41,43,44,51,52,53,54,55,57,58,59,60,64,66,67,71,73,75],behaviour:[2,17,34,38,53],behind:[4,17,28,34,57],being:[2,3,9,11,12,13,14,17,24,32,33,34,35,37,38,40,42,46,51,52,53,54,55,57,59,60,64,66,67,71,72,75],believ:[17,54,55],bell:17,belong:[5,8,11,26,27,29,34,37,39,53,54,57,59,60,63,67,71,75],below:[2,4,5,8,9,10,11,13,14,17,25,26,27,31,34,35,38,40,41,43,51,52,53,54,55,57,59,64,66,71,72,74,75],benaissa:77,benchmark:[17,54],benefici:8,benefit:[13,17,51,57],bengtson:17,benjamin:[11,17,77],benni:17,berlin:77,bernhard:17,bernstein:24,bertholon:17,bertot:[17,24,72],bertrand:17,besid:[3,17,24,34,57],besson:[5,17],best:[13,17,53,54,57,60,71],best_effort:[13,17],beta1:25,beta2:25,beta3:25,beta:[2,11,17,24,55,57,58,64,71,77],betaiota:17,better:[11,14,17,24,51,52,53,57,59,60,64,67,71,72],between:[3,4,10,11,13,14,17,24,25,26,27,29,33,34,38,39,43,44,46,51,52,53,54,57,58,60,64,65,67,71,72,75],bewar:[17,53,55,63,67],beyond:[59,63],bezem:77,bezout_comm:17,bf:[13,17],bfb0037116:77,bfb0040259:77,bformula:5,bg:66,bhat:17,bi:3,bibliographi:25,bibtex:17,bidirect:17,bidirection:[17,25],big:[11,14,17,57,59,71],big_int:17,big_int_z:17,big_prop:57,bigbodi:57,bigger:34,biggest:53,bigint:[17,29,71],bign:17,bignat:[29,71],bignum:[17,53],bigop:57,bigq:17,bigvee_:5,bigwedge_:5,bigwedge_i:5,bigz:[17,53],bij:4,biject:[4,17],bin:[17,53],binari:[3,5,7,11,14,17,24,27,29,37,42,51,53,57,58,60,64,71],binary64:[17,27,36],binary_induct:17,bind:[3,9,10,14,17,24,25,28,32,34,35,37,40,43,44,46,51,54,57,64,66,67,72],binder:[12,13,17,24,25,30,32,34,37,38,40,52,54,55,58,59,63,64,67,75],binder_interp:71,bindir:[17,51],binint:[17,53],binintdef:17,binnat:[17,59],binnatdef:[17,59],binnum:[17,59,71],binop:5,binopspec:[5,17],binpo:[17,59],binposdef:[17,59],binrel:5,bird:6,birkhaus:77,bishop:24,bit0_eqb:59,bit:[2,5,17,27,29,30,34,36,51,53,66,71,75,77],bitvector:17,bitwis:[17,59],blaauwbroek:17,black:[17,29],blacklist:[2,17,59],blah:55,blank:[17,24,29,53],blanqui:57,blaudeau:17,blazi:77,bleed:17,bliss:55,blob:[52,71],block:[2,9,10,14,17,25,29,30,34,37,38,44,46,54,64,65,67],blocktyp:8,blow:17,blowup:17,blue:[29,52],bm:57,bmod:57,bodi:[2,4,6,13,14,17,24,32,35,37,38,41,42,44,51,55,57,58,59,64,72,75],bodin:17,bodo:17,boespflug:77,bogu:8,bohannon:17,bold:66,boldfac:29,boldo:24,book:[17,25],bookkeep:25,bool:[2,4,5,12,13,17,24,27,30,35,36,37,40,41,42,44,46,55,57,58,59,60,71],bool_as_dt:17,bool_as_ot:17,bool_cas:40,bool_choic:[27,59],bool_in_nat:4,bool_ind:[27,40],bool_nat:17,bool_rec:[27,40],bool_rect:[27,40],bool_scop:[17,27,41,71],bool_sind:[27,40],boolean_if_scop:57,boolnot:17,boolord:17,boot:17,border:71,borg:17,boro:17,borrow:17,both:[2,3,4,11,14,17,24,25,26,27,28,29,31,34,37,38,40,42,43,44,46,51,52,53,54,57,58,60,61,64,66,67,73,74],bottom:[3,17,37,46,52,54,55,58,64,71],bottomup:3,bou97:[11,77],boulier:17,bound:[3,5,6,7,10,14,17,24,25,26,27,28,31,32,34,39,41,42,44,46,52,54,55,57,58,59,60,62,64,72],boundari:[17,54],bourk:17,boutilli:17,boutin:[11,24,77],box:[12,17,29,54,71],box_ind:12,box_irrelev:12,box_rec:12,box_rect:12,box_sind:12,boyer:[17,24],brace:[25,44,52,59,71],bracket:[17,24,26,44,54,57,59,66,71,75],braibant:17,brain:17,branch:[2,5,9,17,25,34,40,45,46,55,59,60,66,67,72],brand:17,brandenburg:17,breadth:13,breakag:17,breakpoint:[17,25],breitner:17,bresenham:24,breviti:[42,58,66],bridg:[17,57],briefli:[24,27,57],bring:[17,59],broke:17,broken:[11,17,71],brought:17,brows:[17,25,27,52,57,73],browser:[17,52],bruijn:[17,24,31,33,77],bruno:[11,17,24],brute:[57,64],bs:46,btauto:[17,62],btauto_plugin:[11,27,29,36,57,66],btauto_term:62,buchberg:[7,24,77],buffer:[17,25,35,53],bug:[12,17,24,52,54,66],bugfix:17,buggi:[17,25,33],bugtrack:17,build:[2,5,9,11,14,17,24,25,26,27,32,33,34,37,42,46,51,54,55,57,59,60,63,65,66,67,72,75,76,77],build_:37,build_monad:14,build_monoid:14,build_setoid:42,buildlist:46,built:[2,4,11,17,24,25,26,31,32,34,37,41,42,52,53,54,58,60,61,62,67,71,72],builtin:52,bullet:[8,17,25,34,59,67],bump:17,bunch:[17,57],bundl:17,burden:[3,63],busi:17,button:[8,17,24,52],buys:17,bv2n:17,bvand:17,bvector:17,bveq:17,bvneg:17,bvor:17,bvxor:17,byextend:17,bypass:59,bypass_check:[30,32,34,59],bypass_guard:17,byte_scop:71,bytecod:[12,17,59,64],bytevector:17,c0:[11,59],c1:[17,46,57,67,71],c2:[17,46,57,67,71],c3:[57,71],c4:57,c:[0,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],c_1:[5,26,34,35],c_2:5,c_:34,c_i:[5,34,35],c_k:[26,34],c_m:35,c_n:[34,35],c_pattern:57,c_q:34,cach:[5,12,17],cachan:[17,24],caci:17,caglayan:17,calcul:[24,25,77],calculi:[54,62,77],calculu:[11,14,17,24,25,27,29,31,33,34,35,37,46,54,57,58,62,64,66,67,71,77],call:[2,3,4,5,6,9,11,12,13,14,17,24,25,26,27,28,29,30,31,32,34,35,36,37,39,40,42,44,45,46,51,53,54,57,58,59,60,64,66,67,71,72],callabl:2,callback:[2,17],calvin:17,cambridg:[24,77],came:17,caml:[17,24,75],camlc:53,camldir:17,camlflag:[17,53],camloptc:53,camlp4:[17,24],camlp5:[17,71],camlpkg:[17,53],can:[2,3,4,5,6,7,8,9,10,11,12,13,14,17,24,25,26,27,28,29,30,31,32,33,34,35,36,37,38,39,40,41,42,44,45,46,51,52,53,54,55,57,58,59,60,61,62,63,64,65,66,67,71,72,73,74,75],can_in_comp:17,can_in_pcan:17,cancel:[11,38,41,57,66],candid:[57,58,64,72],cannot:[2,3,4,8,9,10,11,12,13,14,17,26,28,29,32,34,35,36,37,40,41,44,46,51,53,54,55,57,58,59,60,62,64,66,67,71,72,75],canon:[2,4,5,11,13,17,24,25,30,32,34,35,37,38,44,45,53,57,59,71,77],cantor:[17,34],capabl:[3,17,51,53,54,55,64],capit:[17,29,74],captur:[3,17,34,44,57,64,71],car:3,carbonneaux:17,card:57,card_nat:54,cardinal_add_in:17,care:[2,13,14,17,46,53,54,64,67,71,75],carefulli:60,carl:17,carlo:[24,77],carri:17,carrier:[3,11,14,42,57],carst:17,cartesian:[14,54],carthi:60,cascad:17,case_eq:17,case_item:40,case_l_r:17,case_l_r_l:17,case_l_r_r:17,casetyp:17,cast:[2,12,17,25,40,46,54,55,57,58,60,64,71],casual:[25,57],cat:[17,27,74],categor:24,categori:[4,8,13,17,35,51,59,61,74,75],catherin:9,cauchi:[17,27],caught:[46,54,55],caus:[8,12,14,17,32,51,52,53,54,55,57,58,59,63,64,66,71,75],caution:66,caveat:[2,17,25,55,57,60],cbn:[10,17,41,64],cbv:[10,14,17,24,31,57,64],cc:[53,77],cd:[2,17,53],ce:42,ceil:5,cell:36,centaur:24,central:[24,25],centuri:24,cep:17,cequival:3,certain:[4,17,24,29,44,46,51,54,57,58,59,64,67,71],certif:17,certifi:[2,9,17,24,77],cezari:17,cf07:[36,77],cf:[2,9,17,24,29,34,40,42,46,59,67],cfc58:[26,77],ch85:[24,77],ch86a:[24,77],ch86b:[24,77],chailloux:24,chain:[2,17,25,51,64,71,74],chaje:[17,58],challeng:[17,24,77],chalmer:[24,77],chanc:[17,53],chang:[2,4,5,8,9,11,13,14,25,26,28,29,31,34,36,37,38,41,43,51,52,53,54,57,58,59,60,62,63,64,66,67,71,73,74,75],change_arg:17,change_no_check:[17,58,64],changelog:[17,24],changement:24,channel:[17,51],chantal:17,chap:24,chapoton:17,chapter:[2,3,8,9,11,13,15,17,24,26,27,29,31,32,33,34,38,40,42,45,52,54,55,57,58,59,61,63,65,71,73,75,76],char63:[27,36],char_scop:71,charact:[2,8,10,14,17,24,25,27,29,35,36,40,44,46,53,54,55,57,58,59,64,66,71,72,74,75],character:[8,17,34,40,42],characterist:5,charg:17,charset:[52,75],chasl:24,chat:17,chatzikonstantin:17,cheap:17,cheapli:46,check:[2,3,4,5,6,8,9,10,11,12,13,14,17,24,25,26,27,30,32,33,34,35,37,38,39,40,41,42,43,44,46,51,52,53,55,57,58,59,60,62,64,66,67,71,72,74,75],check_guard:59,check_posit:59,check_univers:59,checkabl:24,checkbox:52,checker:[2,9,11,17,24,25,26,29,33,73],checkproof:17,checksum:[17,51],chet:24,chetan:24,chile:17,chines:[2,24],chiron:17,chlipala:17,chluebi:17,cho:17,choic:[3,17,27,34,51,52,55,62,71,75],choice2:27,choicefact:17,choos:[2,3,17,32,34,42,43,52,53,54,57,58,67,71,72,75],chose:53,chosen:[11,34,54,55,57,58,66,71],christian:17,christin:[17,24,27,34,77],christoph:[2,17,24,77],chronolog:15,chung:17,church:[24,77],ci:[11,17,53,57,73],cic:[0,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],circ:27,circular:[4,17,57],circumv:17,cjk:[17,29],clamp:57,claret:17,clarif:17,clarifi:[17,24],clariti:[58,66],clash:[2,17,53,54,57],class_1:17,class_2:17,class_of:42,classic:[11,17,24,25,27,34,51,55,57,66],classical_left:[17,58],classical_prop:17,classical_right:[17,58],classicaldedekindr:17,classicalfact:17,classifi:[17,27],classnam:13,claud:17,claudel:17,claudio:[3,17,24],claus:[9,13,14,17,24,25,28,29,30,32,34,35,40,41,51,53,54,55,57,59,60,62,64,67,71,72],clean:[17,53,57,67,72],cleanal:[17,53],cleaner:17,cleanup:17,clear:[17,24,25,29,38,41,44,54,55,58,64,67,71],clear_switch:57,clearbodi:[17,24,38,58],clearer:55,clearli:[11,24,71,74],clenv_refine_in:17,clerc:17,clever:[17,59,64],click:[8,17,52],client:17,clipboard:52,clock:64,clos_refl_tran:17,clos_t_clos_rt:17,close:[2,3,4,5,7,9,11,14,17,24,28,29,32,34,35,38,44,51,52,55,57,59,60,64,66,67,71,75],closedn:17,closer:[17,24,31,57,60,72],closest:[27,53],closur:[17,24,31,54,55,62,66],club:17,cm:53,cma:17,cmafil:53,cmd:[3,17,38,51,52,54],cmi:17,cmifil:53,cmo:[51,59],cmofil:53,cmorphism:[3,17],cmp:42,cmu:24,cmx:[2,3,5,6,9,11,17,27,29,34,36,42,43,51,54,55,57,58,59,60,64,66,72],cmxa:17,cmxafil:53,cmxfile:53,cmxsfile:53,cn:17,cnet:24,cnr:24,co:[4,10,11,17,24,25,42,44,54,57,59,64,67,71,77],co_high:14,co_low:14,coarser:17,coc:24,coc_histori:17,cockx:77,code:[9,10,11,12,17,24,25,29,33,36,51,52,53,54,55,57,59,60,63,64,71,72,73,74,75],codebas:17,codifi:[55,77],codomain:[17,42,71],coeffici:[7,11,17],coen:[3,17,24],coerc:[4,41,57,60,64],coercibl:[9,57],coercion:[9,13,17,24,25,28,35,37,38,41,42,45,57,58,59,77],coercion_class:[4,71],coexist:17,coffe:17,cofix:[17,25,28,29,31,44,54,55,57,64,67],cofix_bodi:30,cofix_definit:[30,38],cofixpoint:[17,29,30,32,34,38,57,59,64,66],cohen:17,coher:[17,41],coin:5,coinduct:[14,17,25,26,27,32,33,34,37,40,46,59,67,71],collabor:77,collaps:[14,17,51],colleagu:24,collect:[10,17,27,51,53,60,66,72],collid:24,collis:[17,24,51],colog:77,colon:[17,51,53,57,66],color:[8,17,25,51,52,66,75],colson:24,column:[17,46,53,57],com:[2,5,17,51,52,54,71],comand:17,combin:[2,3,5,9,12,14,17,24,25,26,27,29,34,37,40,42,46,52,53,54,55,57,59,63,64,75],combinator:17,combinatori:77,combine_length:17,come:[2,6,8,13,17,24,27,34,43,51,52,54,55,57,59,60,64,71],comextradep:59,comfort:[17,46],comit:17,comma:[17,46,51,52,55,57,74],command:[2,4,5,6,7,8,9,10,11,12,14,16,25,26,27,28,29,30,32,34,36,37,38,40,41,42,43,44,45,46,53,54,55,58,60,62,63,64,72,73,74],commemor:[24,77],comment:[2,5,17,24,25,29,52,54,57,60,66,75],commit:[17,53,54,55],common:[11,14,17,25,26,27,29,31,32,34,42,55,57,60,67,71,74],commonli:[9,14,17,27,40,53,54,55,57,58,66],commun:[2,17,24,27,29,51],commut:[7,11,17,24,44,59],comp:[17,53],compa:17,compact:[17,24,25,34,54,57,59,66,71],compani:[17,66],companion:43,compar:[4,5,11,14,17,24,25,27,37,42,53,54,55,57,58,64,66,67,73],compare_cas:17,compare_cont:17,compare_dec:[17,24],compare_structur:54,comparison:[5,14,17,24,27,42],compat:[2,3,4,13,14,24,25,29,34,42,51,52,53,58,59,62,63,64,71],compatibl:17,compcert:25,compil:[2,3,8,9,10,11,12,24,25,26,27,29,32,35,36,38,46,55,58,64,73,74,75,77],complement:[17,57],complementari:[2,17,24,27,42,57],complet:[3,4,5,6,7,8,9,10,11,17,24,29,30,32,34,36,40,42,51,52,53,54,57,58,59,60,62,66,67,71],completeness_weak:17,complex:[2,11,17,24,25,29,33,35,52,54,55,57,59,61,63,66,67],compli:36,compliant:17,complic:[34,43,46,55],compon:[13,17,24,25,30,33,34,35,37,42,51,52,53,54,57,59,60,71],compos:[3,4,34,44,57,67,71],composit:[3,27,71],compound:[29,54],comprehens:24,compress:[51,53],compris:[3,24],compspec:17,comput:[2,3,7,9,11,17,24,25,27,29,30,32,34,35,36,37,41,42,46,51,52,55,57,59,67,71,72,77],computation:66,con:[0,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],conc:67,concat:[17,46,55],concat_length:17,concat_nil_foral:17,concaten:[17,26,27,54,55,67],concept:[17,24,25,31,57,77],conceptu:[3,34],concern:[2,12,17,24,26],conchon:77,concis:[55,57],concl:[17,59],concl_occ:58,conclud:[5,13,17,34,54,57,64,67],conclus:[3,11,13,17,24,28,34,54,55,57,58,60,64,66,67,71],concret:[2,13,14,17,25,26,29,34,42,46,51,57,64,71],concurr:17,condit:[3,4,9,11,17,24,25,27,30,50,53,59,60,63,64,66,67],cone:[5,17],conejero:17,conf:[17,53],confer:[24,77],confid:[17,24,25],config:[17,51,52],configur:[8,17,24,25,29,40,51,52,59,64,66,73],confin:8,confirm:[59,71],conflict:[17,24,25,46,54,55,71],conflit:17,confluenc:[25,31],conform:17,confus:[4,10,13,17,24,26,29,34,44,46,52,55,57,71],confusingli:[17,58],cong_iff_0:17,cong_iff_ex:17,congr:57,congruenc:[3,12,17,24,25,34,54,62,64,67],congruenceclosur:24,conj:[27,57,58,66,71],conjectur:[17,28,66],conjunct:[3,5,11,17,24,27,34,57,59,60,67,71],conli:27,connect:[17,25,57,62,71],connor:17,conor:[67,77],cons2:34,cons3:34,cons:17,cons_inj_bool:44,cons_inj_nat:44,cons_rlist:17,cons_seq:17,consequ:[17,24,26,29,34,38,39,42,43,44,46,52,57,60],conserv:[2,17],consf:[0,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],consid:[2,3,4,5,9,11,12,13,14,17,24,26,28,29,30,31,34,37,41,42,44,46,52,53,54,55,57,58,59,60,64,67,71,73,75],consider:[3,9,17,37,39,46,64,67,71],consist:[3,4,5,11,13,14,17,24,27,30,31,34,35,52,55,57,58,59,64,65,66,71],consn:46,consol:54,consolid:17,consortium:17,constabl:24,constant:[2,4,5,6,9,10,11,13,14,17,24,25,26,27,30,31,32,34,35,36,38,41,42,44,46,51,54,55,57,58,60,64,66,67,74],constantli:57,constitut:[25,39,55],constr:[3,5,14,17,24,34,42,54,55,57,71],constr_eq:17,constr_eq_nouniv:17,constr_eq_strict:[17,54],constr_may_ev:17,constr_with_bind:17,constrain:[9,14,24,60,67],constraint:[3,5,8,9,10,13,17,24,25,34,35,39,43,44,51,53,54,55,58,67,71],constrast:37,constrexpr:17,construct:[3,4,5,8,9,10,11,13,14,17,25,27,28,29,30,31,33,35,41,42,43,46,52,53,55,57,58,62,63,64,65,66,67,71,77],constructivecauchyr:17,constructiveepsilon:17,constructiveminmax:17,constructivepow:17,constructiver:17,constructor:[2,4,9,10,12,13,14,17,24,25,26,27,30,31,32,35,36,37,40,41,42,43,44,46,54,55,57,58,59,60,62,64,66,71,74],consult:64,consumpt:[8,17,54,55],consw:34,contact:[17,52],contain:[2,5,7,8,10,13,14,15,17,24,27,29,30,31,34,35,38,39,41,42,43,44,46,51,52,53,54,55,57,58,59,60,62,64,66,67,71,72,73,74,75],contains0:67,contains0_ind:67,contains0_sind:67,contant:31,content:[2,17,24,27,32,35,42,51,52,53,54,57,59,66,71,75],context:[4,5,9,10,11,14,17,24,25,26,29,30,31,32,34,35,38,41,43,44,51,52,59,60,62,64,66,67,71],contextu:[17,24,25,31,41],contigu:[17,29],continu:[2,17,24,52,53,54,55,57,71,73],continut:17,contract:[10,17,24,31,34,54,62,71,77],contradict:[17,34,54,57,60,67],contradictori:[17,67],contrainst:17,contrari:[3,4,9,13,17,30,40,44,57,67],contrast:[14,17,34,53,57,60,62,64,67],contrastingli:29,contravari:14,contravariantli:3,contrib:[2,17,24,53,55],contribut:[17,25,53,71],contributor:17,control:[2,3,13,14,16,17,24,25,34,37,41,51,52,53,55,60,62,67,71,75],control_command:[17,29,59],contructor:67,conv:26,conv_expr:17,conveni:[2,4,6,12,17,24,28,29,33,34,35,44,46,52,53,54,57,66,67,71],convent:[2,17,25,33,42,51,57,59,71],convention:[17,53,71],converg:17,convers:[2,3,7,8,9,11,12,13,17,24,25,26,30,32,33,34,35,37,54,55,57,58,60,66,71,75],convert:[3,4,12,13,14,17,25,26,27,34,37,41,44,54,55,57,58,64,67],convert_concl_no_check:17,convinc:24,cook:17,coolen:17,coordin:[17,24],copattern:30,cope:17,copi:[2,17,36,46,52,53,54,57,59,75],coq84:17,coq85:[17,31,77],coq86:[39,77],coq88:17,coq89:[24,77],coq92:[34,77],coq:[2,9,11,13,15,17,25,26,29,30,46,51,53,54,55,57,58,59,63,66,71,72,73,75,76,77],coq_:2,coq_color:[17,51,66],coq_flag:53,coq_makefil:[17,24,25,51,52,59],coq_micromega:5,coq_profile_compon:51,coq_src_subdir:53,coq_vers:53,coqbin:[17,51,53],coqbot:17,coqc:[17,24,25,29,52,54,59,66,75],coqchk:[17,25,53,64,73],coqchkextraflag:53,coqchkflag:[17,53],coqcorelib:53,coqdebug:53,coqdep:[17,25,51,59],coqdev:17,coqdir:[17,75],coqdoc:[17,24,25,51,53,76],coqdocdir:17,coqdocextraflag:53,coqdocflag:[17,53],coqdocid:75,coqdocinstal:[17,53],coqdockw:75,coqdocmodul:75,coqextraflag:53,coqflag:[17,53],coqid:[8,25,35,51,53,54,66,76],coqiderc:[17,52],coqidetop:17,coqlib:[17,51,53,71],coqlib_path:17,coqlib_url:[17,75],coqlibinstal:[17,53],coqmakefil:[17,25,52],coqmakefile_vers:53,coqn:[17,51,53],coqoon:17,coqpath:[17,51,53],coqplugininstal:[17,53],coqpp:[17,53],coqprefixinstal:17,coqprim:17,coqproject:53,coqrc:[24,25],coqremotebrows:17,coqrunbyteflag:17,coqtail:[51,53,66],coqtest_skipcomplex:17,coqtimelog2html:[17,53],coqtoolsbyteflag:17,coqtop:[17,24,25,26,35,52,53,54,59,66],coqtop_toplevel:53,coquand:[24,34,77],coqworkmgr:17,coram:75,corbineau:[17,24],core:[3,13,17,24,25,27,29,41,45,51,53,54,57,59,60,62,65,71],core_scop:[14,71],corecurs:[25,33,71],corn:[24,46,67,77],cornel:24,corner:[17,64],corollari:[17,32],corpu:57,correct:[2,8,9,11,17,24,25,27,28,32,35,46,51,53,57,59,64,66,67,71],correctli:[17,24,29,34,51,52,53,54],correspond:[2,3,8,9,11,13,14,15,17,24,26,27,28,33,34,35,37,38,42,44,46,51,52,53,54,55,57,58,59,60,64,66,67,71,72,75],corrupt:[17,24],cos3pi4:17,coscoi:24,cosin:17,cosmo:77,cost:[17,51,55,60],could:[2,3,4,5,6,11,12,17,24,29,31,34,37,42,46,51,52,55,57,58,60,62,66,71,72,73],couldn:13,count:[13,17,25,51,57,58,59,64,66,67],count_occ:17,count_occ_app:17,count_occ_bound:17,count_occ_elt_eq:17,count_occ_elt_neq:17,count_occ_repeat_eq:17,count_occ_repeat_excl:17,count_occ_repeat_neq:17,count_occ_rev:17,count_occ_sgt:17,count_occ_uniqu:17,countabl:17,counter:[17,62],counterpart:[2,3,9,11,17,27,30,34,57],counterproduct:17,coupl:[11,17,46,53,57,75],courant:24,cours:[2,14,17,24,42,51,52,57,64,71],courtesi:17,courtieu:[17,24],cousineau:24,couterbal:17,covari:14,covariant_ind:14,covariant_rec:14,covariant_rect:14,covariant_sind:14,covariantli:3,cover:[17,44,54,57,65],cp90:[24,34,77],cp:53,cp_phi:11,cpattern:[54,55],cpermut:17,cpow:11,cpp:77,cpu:[17,59],cr_of_q:17,craft:[54,57],craig:77,cran:17,crash:17,crashcoqid:52,creal:17,creat:[3,8,9,13,17,24,25,29,34,38,40,42,51,52,53,54,57,58,59,64,66,67,72,75],creation:[17,24,43,60],credit:[17,24],crelat:3,crelationclass:17,cring:17,cristal:24,cristina:[24,46,67,77],criteria:[2,17,72],criterion:[10,17,33,34,60],critic:[17,24,33,54,59],croap:24,crone:17,cross:[17,24,35,38,64,66,71],cryptograph:24,crzero:17,cs:[17,24],csdp:5,css:[52,75],cst1:17,cst2:17,cst:17,cstop:5,ct95:[67,77],ctan:75,ctcoq:24,ctl:24,ctltctl:24,ctrl:[17,52],ctw21:[10,77],ctx:67,ctx_ind:67,ctx_rec:67,ctx_rect:67,ctx_sind:67,cube:77,culmin:24,cumbersom:[44,55],cumul:[12,13,17,24,25,26,29,30,31,34,37,40,71],cumul_univ_decl:[14,34],cup:[17,26,34,51],cur:54,curiou:5,curli:[8,25,44,59,71],current:[2,3,4,5,8,9,10,12,14,17,24,27,28,29,32,34,35,36,37,38,41,42,44,46,51,52,53,54,55,57,58,59,60,64,66,67,71,75],curri:[17,24,26,66,77],cursor:[17,52,66],custom:[2,3,11,13,17,24,25,27,29,36,53,54,57,59],customiz:17,cut:[14,17,24,25,29,52,57,58,60],cutoff:54,cutrewrit:17,cv:[17,51],cv_infty_cv_0:17,cvc3:17,cvcl:17,cycl:17,cyclic31:17,cyclic:[17,27,64],cyclicaxiom:17,cyprien:17,cyril:[17,29],czajka:17,d0:[67,71],d1:71,d2:71,d:[2,4,5,11,14,17,24,26,34,46,51,52,53,54,57,58,62,67,75,77],d_1:11,d_2:11,d_item:57,d_tactic:57,dabrowski:17,dai:[24,51],daili:55,dalrympl:17,dama:77,dan:[17,24,77],danger:17,daniel:[17,24],danilkin:17,dapprich:17,dark:52,darryl:17,dash:75,data:[17,24,27,34,36,39,53,54,55,57,64,66,77],databas:[3,13,17,25,54,57,62,64],datadir:17,datatyp:[2,17,24,25,26,35,44,46,54,55,57,59,60,67,71],date:[17,24,53],davi:24,david:[17,24,72,77],db72:[26,77],db:[3,17],dc95:[54,77],ddoubl:57,de:[17,24,31,33,59,77],dea:[24,77],deactiv:[9,17,24,25,27,46,59],dead:[24,64],deal:[3,5,8,13,17,24,25,42,46,57,60,64,71,72],debian:17,debug:[2,5,9,13,14,17,24,25,28,52,53,57,58,60,62,64,66,72],debug_univ_nam:14,debugg:[17,24,25],dec:[9,24,46],dec_int_scop:[17,71],dec_uint_scop:[17,71],decad:17,decemb:[17,24,77],decentr:17,decid:[5,8,11,17,24,25,27,29,34,51,53,55,57,60,71],decidableclass:17,decidabletyp:17,decim:[5,17,27,29,59,71],decimalfact:17,decimaln:17,decimalnat:17,decimalpo:17,decimalstr:17,decimalz:17,decis:[2,17,24,25,58,62,64,77],decl_not:[30,34,40,71],declar:[2,4,5,6,7,8,9,10,11,12,14,17,24,25,26,27,28,29,30,31,32,34,35,36,37,43,46,51,53,54,58,59,60,64,71,72,75],declareunicodecharact:75,decnat:29,decod:17,decompos:[24,57,67],decomposit:57,deconstruct:46,decor:[24,29,42],decoupl:[8,17],decreas:[3,7,9,17,30,34,55,59,72],decrement:[17,54],dedekind:17,dedic:[11,17,24,29,36,55,57],deduc:[5,17,44,51,57,58,67],deduct:[5,24,57],deem:[2,51],deep:[17,24,57,67],deep_tupl:46,deepen:13,deeper:[34,46],def:[26,35,67],def_bodi:[4,32,38,42],def_n:57,default_bindings_src:52,default_go:53,default_with:17,defaultrel:3,defect:[25,55],defend:24,defens:[17,24,44,57],defer:[52,55,57],defin:[2,3,4,5,6,7,9,11,12,13,14,17,24,25,26,27,28,29,30,31,32,33,36,38,39,40,41,42,43,44,46,51,52,53,57,58,59,62,64,66,67,71,72,74,77],defined:3,definin:35,definit:[2,4,8,10,11,13,17,24,25,26,27,28,29,31,33,35,36,38,41,42,43,44,51,53,58,59,60,62,66,67,72,73,74,75,77],definition:[4,12,17,31,32,35,37,64],definitionalclass:17,degener:[40,57],degrad:54,degre:[5,73],del00:[54,77],delahay:[24,77],delai:[14,17,25,40,64],deleg:[8,17,25,29],delet:[17,52,54,57,66],delete_on_error:17,deliber:[31,55],delic:34,delimit:[8,17,33,35,41,44,59,66,71,75],deliv:17,delpath:[17,24],delphin:77,delta:[11,17,24,32,35,37,55,64],delta_reduct:[55,64],demand:57,demonstr:[24,54,67],dempski:17,denomin:[11,17,37,71],denot:[3,4,11,17,24,26,28,29,30,34,35,39,40,42,43,52,54,57,58,67,71],denum:11,dep:51,dep_ret_typ:46,depart:3,departur:55,depend:[2,3,7,8,9,12,13,14,24,25,26,27,28,29,30,32,34,35,36,37,38,40,42,43,44,51,52,54,55,57,60,62,64,66,71,72,77],deplaix:17,deploi:17,deprec:[2,4,13,17,25,28,29,32,35,41,51,55,58,59,60,64,66,71,72],depth:[3,5,13,17,29,54,57,58,59,60,62,64,71,75],der:17,derek:77,deriv:[3,5,9,13,17,24,25,26,27,30,34,38,40,54,64,66,73],derive_plugin:6,desarzen:17,describ:[2,3,4,6,7,8,10,11,12,13,14,17,24,27,29,31,32,34,35,36,37,39,40,42,43,46,51,52,53,54,55,57,58,59,64,65,66,67,71,72,75],descript:[17,24,25,27,29,31,38,40,42,46,51,53,57,66,67],design:[2,8,11,17,24,25,37,44,57,64,71,77],desir:[9,11,17,34,52,53,54,57,59,73,75],desktop:17,desmettr:[17,24],despit:[36,57],dest:[4,17],destauto:[17,67],destdir:[17,53],destko:17,destroi:55,destruct:[2,13,17,24,25,34,54,55,57,58,64,71],destruct_bool_and_rewrit:54,destruct_with_eqn:71,destructor:[17,25,30,31,37],destructur:[17,24,25,32,40],destructuring_let:[32,46],desugar:37,detach:[17,52],detail:[3,5,7,14,25,27,31,36,37,41,42,51,52,55,57,58,59,64,66,71,72,74,75],detect:[5,8,17,25,41,44,52,53,57,66],determin:[4,13,17,31,34,36,40,41,43,53,54,57,58,64,66,67,71,72,75],determinist:17,dev:[17,24,51,53,71],develop:[2,3,12,13,14,17,24,25,27,32,35,42,44,51,52,53,54,57,58,59,60,64,66,67,71,74,77],devis:17,devot:[52,57],df:[13,17,60],dfrac:5,di:[54,77],diagnos:14,diagnost:71,diagon:34,diagram:11,dialect:17,dialog:[17,52,65],dialogu:55,did:[8,11,17,26,29,57,58,59,66,67],didn:[3,17,51,53],diff2:77,diff:[17,24,25,51,53,54],diff_failur:17,differ:[3,4,9,11,13,14,15,17,24,25,26,27,29,31,34,35,37,38,41,43,46,51,52,53,54,55,57,58,59,60,62,64,67,71,72,73,75,77],difficult:[11,17,29,55,71,72],difficulti:53,digit:[17,24,27,29,44,51,52,71],dimens:17,dintuit:[17,62,71],dir:[17,51,53,75],direct:[2,9,12,16,17,24,31,34,42,46,52,53,57,58,59,71],directli:[2,3,4,9,13,14,17,24,27,28,34,43,51,52,53,55,57,58,59,60,64,67,72,75],directori:[2,14,17,24,27,35,51,52,53,59,60,71,75],dirpath:[17,35,51,59],disabl:[2,8,9,12,13,14,17,25,28,32,34,35,37,44,51,52,54,57,58,59,64,66],disallow:[12,14,17,37,51],disambigu:[17,44,57,71],disappear:[2,17,24,34,55,60,67,71],discard:[14,17,52,54,55,58,64,75],discharg:[3,14,17,24,25,28,38,72],disciplin:[17,24,26],discontinu:17,discourag:[17,29,32,35,53,54,55,58,59,60,66],discours:[17,52],discov:[17,53],discoveri:24,discrep:[17,57],discret:5,discrimin:[13,17,24,54,57,58,59,60,62,64,66],discrimine:[10,12,46],discrr:[24,27],discuss:[3,17,24,25,54],disembodi:42,disequ:[9,60],disj:[17,71],disjoint:[27,67],disjointed:67,disjunct:[17,25,34,57,58,59,60,67,71],disk:[51,52,53,66],dismiss:67,dispatch:55,displai:[2,9,12,14,16,17,25,35,37,41,42,46,51,53,54,55,57,58,60,64,66],dispos:57,disregard:42,distanc:24,distinct:[9,13,17,26,34,42,44,46,53,54,55,57,60,64,67,71],distinguish:[14,17,24,26,34,37,57,64,71],distr:2,distribut:[11,17,24,25,50,73,75],disus:17,div0:[17,59],div2:[9,17,72],div2_0:17,div2_1:17,div2_decr:17,div2_equ:72,div2_even:17,div2_ind:72,div2_l:72,div2_le_lower_bound:17,div2_le_mono:17,div2_le_upper_bound:17,div2_obligation_1:9,div2_obligation_2:9,div2_obligation_3:9,div2_obligation_6:9,div2_odd:17,div3:9,div:[2,3,5,11,17,27,59],div_exact:59,div_mod:17,div_mod_to_equ:[5,17],div_theori:11,div_zdiv:17,diveq_iff:17,diveucl:2,divex:2,divid:[5,15,17,24,58],divide_gcd_iff:17,divide_to_equ:5,divis:[3,11,17,24,25,57],divisor:[7,17],dj:57,dm82:[55,77],dmitri:17,do_depind:67,do_makefil:24,doc:[17,24,51,53,63,71,74,77],doc_grammar:17,docdir:[17,53],docgram:71,docker:17,docroot:[17,53],doctor:24,doctorat:77,document:[3,8,9,11,12,16,17,24,25,27,42,51,52,54,55,57,59,64,65,66,67,71,72,74,76],doczkal:17,doe:[2,3,4,5,8,9,12,13,14,17,24,25,26,27,29,30,34,35,36,38,39,41,42,44,51,52,53,54,55,57,58,59,60,62,64,66,67,71,72,75],doesn:[4,14,17,27,29,31,35,46,51,52,53,54,55,57,58,59,62,66,67,71,73],doi:77,doligez:24,dom:71,domain:[3,5,11,14,17,24,25,26,34,42,61,64,71],domin:75,dominiqu:17,don:[4,10,13,14,17,28,34,35,37,46,52,53,54,57,58,60,62,64,66],donati:17,done:[2,3,5,6,7,9,10,11,13,17,24,27,29,30,32,34,35,36,38,40,42,43,46,52,53,54,55,57,58,59,60,64,66,67,71,72,75],dont:[17,59],dorel:17,dot:[11,14,17,24,35,37,52,59,71],doubl:[17,24,27,29,34,44,52,53,54,57,59,71,75],double_var:17,doublen:57,dowek:24,down:[3,14,24,25,45,51,52,54,55,57,59],download:[17,27,53,77],dozen:64,dp:[2,17],drag:[17,24],dramat:64,draw:24,drawback:[9,17,67,71],dreyer:77,drive:64,driven:[24,60],driver:5,drop:[3,17,51,54,59,71],drope:17,dstroot:17,dt:60,dtauto:[17,62],dual:[3,9,24,55],dualli:[3,44,57],duboi:17,dudenhefn:17,due:[2,3,13,14,17,24,27,30,34,46,52,54,55,59,64,66,67,71,72,73],dummi:[2,14,17,24,55,77],dummy_ind:14,dummy_rec:14,dummy_rect:14,dummy_sind:14,dump:[5,17,24,51,75],dumpbox:17,dumpgraph:17,dune:[17,25,51,59],dup:[17,57],duplic:[3,11,17,43,57,67,71],duprat:24,durat:51,dure:[2,9,11,13,14,17,24,37,42,46,51,53,54,55,57,58,60,64,66,67,71,72],duti:55,dvdn1:57,dvdn_mull:57,dvdn_mulr:57,dvdn_subr:57,dvdn_tran:57,dvi:75,dx:77,dyc92:[54,62,77],dyckhoff:[24,54,62,77],dynam:[2,11,13,17,25,36,51,59,71],dynlink:[17,59],e0:[42,46,72],e1:[17,42,46,57],e2:[17,42,46],e:[0,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,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],e_1:[5,35],e_2:[5,35],e_:[17,35],e_i:35,e_n:35,e_type_of:17,ea:13,each:[2,3,5,6,8,9,10,11,13,14,17,24,26,27,29,30,34,35,36,37,38,39,40,42,43,44,46,51,52,53,54,55,57,58,59,60,64,66,67,71,72,74,75],eager:17,eagerli:55,eappli:[17,54,58,60,66,67,71],earli:[2,15,17,25,26,54,64],earlier:[8,17,53,54],eas:[13,17,37,53,55,57,58,66],easi:[7,11,13,17,27,46,52,53,60,67],easier:[2,10,17,24,45,52,57,58,67,71],easiest:53,easili:[13,17,53,57,72],eassert:[17,43,58],eassumpt:[17,43,58,60],eauto:[17,25,43,54,57,60],eb:13,ecas:[17,43,58,67],echo:53,econom:[24,77],econstructor:[17,43,67],ecosystem:[25,73,77],ed:[17,24],edestruct:[17,43,58,67],edg:[17,52],edinburgh:24,ediscrimin:[17,43,67],edit:[17,24,25,29,51,53,57,66,71],editor:[17,52,53,77],eduardo:24,edward:17,eelco:77,eeli:17,eelim:[17,43,67],eenough:[17,43,58],eexact:[17,43,58],eexist:[17,43,60,66,67],effect:[2,9,11,13,14,17,24,25,29,30,34,35,38,43,51,52,53,54,57,59,64,66,71,75],effici:[2,11,12,13,17,25,29,36,57,60,64,77],effort:[13,17,24,63,74],eg:[17,53],ei:57,eight:34,einduct:[17,43,58,67],einject:[17,43,67],eintro:[43,58],either:[2,5,8,11,14,17,26,28,29,31,34,35,36,37,39,40,41,44,46,51,52,53,54,55,57,58,59,60,64,66,67,71,74,75],ej:57,el:77,elabor:[13,14,17,25,27,33,37,41,44,45,51,55,58],elaps:54,elast:24,elect:[25,50],electron:[24,77],eleft:[17,43,67],eleg:[2,55,59],elegantli:58,element:[2,3,11,12,17,25,26,27,34,35,36,46,57,59,60,71],elementari:[25,27,57,58,71],elements1:71,elements2:71,elid:57,elim:[5,17,24,25,54,58,67],elim_let:17,elimin:[10,12,14,17,24,25,26,27,30,31,34,35,37,40,54,55,58,67,71,72,77],elimtyp:17,elpi:[17,63],elrod:17,els:[2,4,9,11,12,13,17,29,30,35,40,41,46,52,54,55,57,62,67,71,75],elsevi:77,elsewher:[9,17,52,59,71],elt:5,elt_eq_unit:17,emac:[17,51,52,59,66],email:52,emb:[17,24,71],embed:[24,25,29,71],emerg:24,emilio:17,emit:[2,10,12,13,17,34,53,71,74],emmanuel:24,emp:60,emphas:46,emphasi:25,emploi:[17,42],empti:[2,3,5,7,12,13,17,24,26,34,40,43,51,53,55,57,58,59,60,67,71,72],empty_context:17,empty_neutr:3,empty_set:[17,40,62,71],emptyf:[0,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],emul:[2,12,17,40,57],en:[24,57,64,77],enabl:[2,4,7,8,9,10,11,12,13,14,17,25,34,37,42,51,52,53,54,57,58,59,60,67,75],enable_notation_flag:71,encapsul:57,enclos:[2,29,41,53,54,55,66,71,75],encod:[3,13,17,24,25,27,34,53,71,75],encount:[2,11,17,52,53,54,64],encourag:[17,46,53,54],end:[0,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,35,36,37,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],enforc:[9,12,14,17,26,32,34,44,55,57,58,66,71],engin:[13,17,24,33,43,55,57,58,64,77],english:17,enhanc:[2,17,52,57],enjoi:[31,34,37,57],enough:[10,11,14,17,34,44,57,58,67,71],enrich:[5,17,24,26,27,67],enrico:[8,17,42,57,77],ensur:[2,10,13,14,17,24,27,30,34,39,52,55,59,64,71,72],ensuremath:75,enter:[8,17,25,30,32,34,35,38,44,46,52,54,55,59,60,71],entier:17,entir:[10,13,17,24,25,31,33,34,41,44,52,53,57,60,64,66,71],entri:[17,24,25,28,29,37,51,52,53,54,55,67],enumer:[5,17,34,40],enviro:[17,59],environ:[3,9,11,12,13,14,17,24,25,26,28,30,31,32,34,35,38,42,43,52,53,55,57,60,62,64,66,67,71,72,75],envr:5,ep:60,epos:[17,43,58,71],epsilon:[17,60],epsilon_smallest:17,eq0:3,eq0_le0:44,eq:[3,5,11,14,17,27,35,40,42,54,57,58,59,64,67,71],eq_:27,eq_add_:27,eq_adda_b:57,eq_adda_c:57,eq_big:[17,57],eq_big_:57,eq_bigr:57,eq_bigr_:57,eq_bool:13,eq_class:42,eq_dec:17,eq_ex2:17,eq_ex2_hprop:17,eq_ex2_uncurri:17,eq_ex:17,eq_ex_hprop:17,eq_ex_intro2:17,eq_ex_intro2_hprop:17,eq_ex_intro2_uncurri:17,eq_ex_intro:17,eq_ex_intro_hprop:17,eq_ex_intro_uncurri:17,eq_ex_uncurri:17,eq_ind:[14,27,40],eq_ind_r:[11,27],eq_izr_contraposit:17,eq_map:57,eq_mod_ab:17,eq_mod_opp:17,eq_nat:[24,42],eq_nat_dec:17,eq_nat_equiv:42,eq_pattern:17,eq_rec:[14,27,34,40],eq_rec_r:27,eq_rect:[14,17,27,34,40,67],eq_rect_r:[17,27],eq_refl:[5,9,11,12,13,14,17,27,40,57,64,66,67,71],eq_reflex:59,eq_rel:3,eq_rel_reflex:3,eq_rel_rel:3,eq_rel_symmetr:3,eq_rel_transit:3,eq_set:3,eq_set_refl:3,eq_set_rel:3,eq_set_rel_reflex:3,eq_set_rel_rel:3,eq_set_rel_symmetr:3,eq_set_rel_transit:3,eq_set_sym:3,eq_set_tran:3,eq_sig:[17,67],eq_sigt_rect:17,eq_sind:[14,27,40],eq_sym:[27,40,44],eq_symmetr:59,eq_tran:[27,59],eq_trans_assoc:59,eq_tru:17,eq_true_is_tru:12,eqa:[3,13],eqab:57,eqac:57,eqb0:57,eqb:[3,5,13,17,27,36,59],eqb_correct:36,eqb_leibniz:13,eqb_sym:59,eqba:57,eqblr:17,eqbrl:17,eqca:57,eqd0:57,eqdec:[13,38,60],eqdec_def:13,eqdep:17,eqdep_dec:[17,67],eqlista:17,eqn:[17,40,55,57,58,67,71],eqn_mul1:57,eqnarrai:34,eqnat:[17,26,42],eqnot:17,eqo:3,eqp:57,eqst:30,eqst_hd:30,eqst_tl:30,eqt:[17,46],eqt_ind:46,eqt_rec:46,eqt_rect:46,eqt_sind:46,equal:[3,5,8,10,11,12,13,14,17,24,25,26,30,31,32,34,35,36,39,40,42,44,46,52,54,55,57,58,60,61,65,71,72,77],equalitiesfact:17,equality_intropattern:58,equat:[5,6,14,17,24,25,27,34,40,42,46,53,55,58,60,61,64,67,72],equations_plugin:53,equiconsist:34,equip:[3,4,17,24,27,36,42,64],equiv:[5,34,39],equival:[3,9,11,12,13,14,17,24,25,26,27,28,29,32,34,35,36,37,38,41,42,46,51,52,53,54,55,59,60,62,64,66,67,71,75],equivalence_class:64,equivalence_reflex:[3,59],equivalence_symmetr:[3,59],equivalence_transit:3,equivlista:17,eras:[17,44,57,58,67,75],erasur:[58,67],erbsen:17,erememb:[17,43,58],erewrit:[17,43,64],ergo:17,eright:[17,43,67],erik:17,erika:17,err:[42,55],erron:17,error:[2,3,4,9,10,11,12,13,14,16,17,24,25,27,28,29,32,34,35,37,38,39,40,41,42,44,46,51,52,53,57,58,59,60,62,64,66,67,71,72,75],es:10,esc:17,escap:[12,17,25,51,53,71],eset:[17,43,58],eshkeev:17,esimplifi:67,esimplify_eq:[17,43],especi:[7,15,17,24,26,34,44,46,54,57,60,62,64,71],esplit:[17,43,67],essai:77,essenti:[2,17,25,34,55,57,67,71],establish:[3,17,57],estim:74,et:[3,24,77],eta:[13,17,25,31,37],etc:[2,4,9,14,17,24,25,26,27,33,35,42,44,45,51,52,53,54,55,57,59,71,75],etcdir:17,eth:17,ethan:17,etransit:[3,17,43,64],eucl_dev:2,euclid:[2,17,24],euclid_intro:17,euclid_rec:17,euclidean:[11,17,24,25,57],euclidean_division_equations_cleanup:[5,17],euclidean_division_equations_find_duplicate_quoti:5,euclidean_division_equations_flag:17,eugen:77,european:[24,77],ev:58,eval:[3,5,12,14,17,24,25,27,29,30,31,32,35,37,42,52,53,55,59],eval_bf:5,eval_earli:54,evalu:[2,3,9,11,17,24,25,28,30,34,35,41,53,57,60,64,71],evar:[17,24,54,55,57,58,59,64,71],evarconv:17,evarmap:17,even:[0,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,68,69,70,71,72,73,74,75,76,77],even_0:34,even_:34,even_alt:17,even_alt_even:17,even_even:17,even_ind:[34,67],even_o:34,even_odd:[17,67],even_odd_ind:17,even_sind:[34,67],even_ss:34,eveno:[0,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],event:[2,17,51],event_oddt_dec:17,event_oddt_rect:17,eventu:[5,17,34,42,43,52,54,55,57,58,60,66],ever:[17,52,55,57,67,71],everi:[3,9,11,12,13,14,17,28,29,34,40,51,52,54,55,57,58,64,71],everybodi:17,everyth:[2,17,52,53],everywher:[2,17,55,58,64],evgeni:[5,17],evgenii:17,evolut:[17,77],evolv:[17,24,37,52,54],ex1:55,ex2:[17,24,27,55,67],ex2_ind:27,ex2_sind:27,ex:[3,17,24,27,44,58,67,71],ex_ind:27,ex_intro2:27,ex_intro:[27,37,41,57,60,66],ex_sind:27,exact:[3,12,14,17,24,25,35,40,43,53,54,55,58,59,60,64,66,67,71],exact_no_check:[58,66],exactli:[4,10,11,13,17,26,27,34,40,42,44,46,51,52,54,55,57,59,66,67,71],exactly_onc:25,examin:[46,52,54,66,67,71],exampl:[7,8,9,13,24,25,32,36,45],example_lra:5,example_map:57,exc:[24,27],exce:[59,67],excel:17,except:[2,3,4,11,12,13,14,17,24,25,26,27,29,31,34,35,36,38,40,43,51,52,53,54,57,58,59,60,64,66,67,71,75],exception:[17,24,64],excerpt:36,excess:24,exchang:[24,52,66],exclud:[17,34,41,51,53,54,55,57,59],exclus:[29,57],execut:[6,17,24,25,29,36,51,52,53,55,57,59,64,66,67,71],exempl:24,exfalso:[17,58],exhaust:[17,29,46,53,54,55,59],exhibit:5,exist2:27,exist:[3,4,5,9,11,13,14,17,25,26,27,28,29,31,32,34,36,37,39,41,42,46,51,52,53,54,55,57,58,59,60,63,64,66,67,71,74],existenti:[3,6,9,10,13,17,24,25,26,34,41,45,54,58,59,60,64,66,67],exists2:[17,27,29,57],exists_app:17,exists_concat:17,exists_differ:71,exists_flat_map:17,exists_fold_right:17,exists_foral:17,exists_map:17,exists_non_nul:71,exists_nth:17,exists_or:17,exists_or_inv:17,exists_rev:17,existt2:27,existt:[17,27,67,71],exit:[8,17,25,30,32,34,38,51,52,54,59,60,75],exn:55,exp:57,exp_ineq1:17,exp_ineq1_l:17,exp_intro:34,expand:[2,13,14,17,28,29,30,31,35,37,41,46,52,54,55,57,58,64,67,71],expans:[10,12,13,17,25,34,53,55,57,64,71],expect:[2,3,4,11,12,14,17,24,26,29,31,32,33,34,40,41,42,43,44,46,51,52,54,55,57,58,60,64,67,71],expens:[13,17,54,66],experi:[17,24,51,77],experienc:66,experiment:[5,10,12,14,17,24,51,53,54,62,66,67,71,72],expert:53,expir:24,explain:[8,13,17,24,29,42,51,52,57,60,71,72,74],explan:[3,13,37,45,51,58,59,67],explicit:[9,10,13,17,24,25,28,31,34,37,39,41,46,55,58,60,64,66,67,71],explicit_id:71,explicit_subentri:71,explicitli:[2,4,12,13,14,17,24,27,28,29,34,38,39,43,46,51,52,53,55,57,58,59,60,64,66,67,71,74],exploit:[3,17,24,57,67],explor:[5,17,59],explos:17,expn:57,expon:[11,17,29,71],exponenti:[5,17,29],expos:[2,17,25,40,41,57,71],exposit:17,expr1:54,expr:[17,54,55,71],expr_0:17,expr_1:17,expr_i:17,expr_ind:71,expr_n:17,expr_rec:71,expr_rect:71,expr_sind:71,express:[2,3,4,5,9,10,11,14,17,24,25,26,27,28,29,30,31,32,34,35,39,40,41,43,44,57,58,59,60,64,66,67,75],exprop:34,exprop_ind:34,exprop_sind:34,expung:24,exs_intro:34,exset:[26,34],ext2:[17,24],ext4:51,ext:[17,24,34],ext_intro:34,extend:[3,4,5,9,10,11,14,17,24,25,26,27,28,29,32,34,35,37,40,41,42,45,51,52,53,55,59,60,71,77],extens:[6,9,10,11,12,14,17,25,26,29,32,41,42,52,53,59,62,63],extension:[12,17,27,30,57],extent:[17,71],extern:[2,5,11,13,17,29,33,52,54,55,59,60,63,66,73,74,75],extgcd:17,extocamlnativestr:17,extra:[8,9,17,24,25,30,34,41,42,46,53,54,57,62,64,66,71,75],extra_reifi:17,extra_scop:17,extract:[9,25,26,27,29,34,36,51,53,57,59,71,72,73,77],extraction2002:77,extraction_plugin:[2,9,34,57,72],extractor:[17,24],extran:[17,52],extrem:[14,17,29,57],extrhaskellbas:17,extrhaskellstr:17,extrocaml:17,extrocamlbigintconv:17,extrocamlfloat:36,extrocamlint63:[17,36],extrocamlintconv:2,extrocamlnatbigint:17,extrocamlnatint:2,extrocamlnativestr:17,extrocamlparrai:36,extrocamlpstr:36,extrocamlstr:17,extrocamlzbigint:17,extyp:34,extype_ind:34,extype_rec:34,extype_rect:34,extype_sind:34,f0:[34,57,67],f10:52,f11:52,f1:[13,17,41,51,57,71],f2:[17,41,51,52,55,57],f4:52,f8:52,f9:52,f:[0,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],f_1:[11,34],f_1_neq_0:11,f_2:[11,34],f_:24,f_equal2:27,f_equal2_plu:59,f_equal3:27,f_equal4:27,f_equal5:27,f_equal:[17,27],f_equalx:17,f_ext:27,f_i:34,f_impl:2,f_ind:58,f_inj:34,f_j:34,f_k:34,f_l:34,f_n:34,f_r:11,f_rec:58,f_rect:58,f_scope:71,f_sind:58,fabian:17,face:[3,17,75],facil:[13,17,24,52,54,55,57,59],facilit:[17,51,57],fact:[2,5,11,14,17,24,28,32,34,39,41,42,46,54,55,57,58,62,64,66,67,71,75],factor:[2,5,11,17,25,34,45],factori:[17,24,54,55,64],factoriz:[17,46],fail:[2,3,4,5,8,9,10,12,13,14,17,24,25,26,29,30,34,35,40,41,42,43,44,52,53,55,58,59,60,62,64,66,67,71,72,75],failur:[3,8,13,14,17,24,25,46,53,55,57,59,60,62,64,71,77],fairli:[17,57],faithful:17,faithfulli:13,fake:60,fall:[3,9,10,13,24,53,58],fals:[2,4,5,9,10,12,13,17,24,27,34,37,40,41,43,46,51,54,55,57,58,59,62,64,66,67,71],false_rec:27,false_rect:46,falsiti:54,falso:[17,58],famili:[4,14,17,24,25,34,40,54,55,63,67,71],faq:17,far:[11,24,46,52,57,66,71],farka:17,farzon:17,fashion:[17,24,51],fast:[3,17,24,25,53],fast_:17,fast_integ:17,faster:[11,17,24,51,58,59,62,64],fastest:53,fatal:[17,25,57],fault:[2,24,71],favor:[17,41,51],fcomp:41,fct:4,fct_of_incr_fct:4,fd:34,fdiv_def:11,fear:33,featur:[2,3,8,11,17,24,25,29,32,33,35,36,44,46,51,52,53,54,55,57,59,66,71,72,73,74,76],feb:24,februari:[17,24],fed:[9,17,55],feed:60,feedback:[8,17],feel:52,feferman:24,fehrl:17,fei:77,felti:24,feq:27,fermat:52,fernandez:17,fernando:17,fetch:66,few:[2,3,17,24,27,29,34,35,36,37,51,52,53,55,57,58,71,73,75],fewer:[17,51,58,64,66],ff:5,ffi:[17,25,55],fg:4,fgt:27,fi:13,field:[4,5,7,12,13,14,17,24,25,27,42,51,53,55,59,61,74],field_mod:11,field_simplifi:17,field_simplify_eq:17,field_spec:37,field_theori:11,field_val:[13,37],fieldnam:37,fifth:17,figur:[52,57],file1:[52,53],file2:[52,53],file:[2,3,5,6,7,8,9,11,17,24,25,27,29,34,35,36,41,42,43,54,55,57,58,60,64,66,71,72,73,76],filen:52,filenam:[14,17,25,51,52,59,64,75],filesystem:[53,59],fill:[2,9,13,17,25,52,55,57,62,71],filliatr:[24,77],filter:[13,17,30,51,53,59,60],filter_2_4:46,filter_app:17,filter_fals:17,filter_length:17,filter_length_forallb:17,filter_length_l:17,filter_map_swap:17,filter_rev:17,filter_some_square_corn:46,filter_tru:17,filtered_import:[17,35,59],filteropt:51,fin:[17,71],fin_scop:71,find:[2,3,4,5,7,11,13,14,16,17,25,27,29,34,42,43,51,52,53,54,55,57,58,59,62,64,66,67,71,72,77],find_duplicate_quoti:17,findlib:[17,53,59],fine:[17,41,51,52,57,64],finer:[2,17,34,57],finfun:17,finish:[8,13,17,29,46,54,60,64,66,67],finish_tim:[17,54],finit:[3,5,17,24,27,30,34],finite_alt:17,finite_dec:17,finv_l:11,fire:[2,14,17],firefox:52,first:[2,4,5,6,8,9,11,13,14,15,17,24,25,26,27,35,37,38,40,41,42,43,44,51,52,53,55,58,59,60,62,64,65,66,67,71,72,74,75,77],first_lett:29,firstn:17,firstn_length:17,firstord:[17,29,62],fissor:17,fit:[14,17,27,29,34,52,55,57,71],five:[17,27,64],fix:[0,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,32,33,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],fix_decl:[34,57],fix_definit:[34,38,72],fix_eq:[17,27],fix_f:27,fix_f_eq:27,fix_f_inv:[17,27],fixabl:17,fixannot:[9,34,72],fixpoint:[2,3,10,13,17,24,25,27,29,30,31,32,37,38,41,44,46,52,57,59,64,66,67,71,72],fk:57,flag:[2,4,5,8,9,10,12,13,14,16,24,25,27,32,34,35,37,38,40,41,43,44,46,51,52,53,54,55,57,58,60,62,64,66,67,71],flagship:25,flambda:17,flat_map:[17,24,27],flat_map_app:17,flat_map_constant_length:17,flat_map_ext:17,flat_map_length:17,flatten:17,flavor:[17,37,71],fledg:17,flexibl:[14,17,55,58,64],flh:5,flip:[3,17],float64:36,float64_mul:36,float64_typ:36,float_class:27,float_comparison:27,float_scop:[27,36],floataxiom:17,floatlemma:17,floatop:[17,36],flocq:27,floor:17,florath:17,florent:17,florin:17,flow:25,flt:27,fly:[17,55,57],fm:13,fmap:[17,60],fmapavl:17,fmapfullavl:17,fmapintmap:17,fn:51,fnotcompar:27,fo:2,focu:[17,24,34,43,54,55,57,66,67],focus:[6,17,25,43,55,57,58,59,60],fof:14,fold:[3,17,37,57],fold_left2:17,fold_left:[17,27],fold_left_length:17,fold_left_rev_right:17,fold_left_s_o:17,fold_right2:17,fold_right:[17,27],fold_right_shiftin:17,foldabl:17,folder:[17,52,53],follow:[2,3,4,5,6,8,9,11,12,13,14,17,24,25,26,27,28,29,30,33,34,35,36,37,38,40,41,42,43,46,51,52,53,54,55,57,58,59,60,62,64,66,67,71,72,74,75],fondamental:77,font:[17,52,53,75],foo0:[53,55],foo1:53,foo:[2,11,14,17,29,35,38,40,43,51,52,53,55,57,58,59,64,66,71,74,75],foo_ind:[12,17,57],foo_rec:17,foo_rect:17,foo_sind:12,foo_subproof:38,foobar:14,foolib:17,footnot:[11,38,57,71],footprint:17,fop:5,for_all2:17,for_each_go:[54,55,71],foral:[2,3,4,5,6,7,9,10,11,12,13,14,17,25,26,27,29,30,31,32,34,36,37,41,42,43,44,46,52,54,55,57,58,59,60,62,64,66,67,71,72,75],forall2:17,forall2_append:17,forall2_cons_iff:17,forall2_flip:17,forall2_impl:17,forall2_length:17,forall2_nil:17,forall2_nth:17,forall2_nth_ord:17,forall2_refl:17,forall_and:17,forall_and_inv:17,forall_app:17,forall_append:17,forall_concat:17,forall_cons_iff:17,forall_elt:17,forall_eq_repeat:17,forall_exists_exists_forall2:17,forall_flat_map:17,forall_fold_right:17,forall_foral:17,forall_imag:17,forall_impl:17,forall_map:17,forall_nil_iff:17,forall_nth:17,forall_nth_ord:17,forall_rev:17,forall_shiftin:17,forallb_filt:17,forallb_filter_id:17,forbid:40,forbidden:[12,17,24,25],forc:[4,8,11,17,24,34,42,44,52,53,54,57,60,64,66,67,71],force2:71,ford:17,foreground:66,foreign:[2,17],forese:24,forest:[0,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,68,69,70,71,72,73,74,75,76,77],forest_ind:[34,67,72],forest_rec:[34,67,72],forest_rect:[34,67,72],forest_s:[34,72],forest_sind:[34,67,72],forest_size_equ:72,forest_size_ind2:72,forest_size_ind:72,forest_size_rec:72,forest_size_rect:72,forest_tree_ind:67,forest_tree_rec:67,forest_tree_rect:67,forg:51,forget:[4,11,37,55,59,60,67],forgot:[32,71],forgotten:4,fork:17,form:[2,3,4,5,6,7,9,11,13,17,24,25,26,27,28,29,30,31,32,35,37,38,39,40,42,43,44,46,51,52,53,54,55,57,58,59,60,62,64,66,67,71,72,75],formal:[4,6,10,17,24,25,26,29,31,32,34,37,39,41,51,55,57,67,77],formalis:[24,57,77],format:[14,17,24,26,27,35,37,42,51,52,53,57,71,75],formatt:59,formel:24,former:[17,29,30,57,75],formerli:17,formul:[17,42],formula:[5,7,26,57,58,62,77],forster:17,forth:[25,50,57,60],forthcom:17,forum:17,forward:[17,24,52,53,57,62,66],found:[2,4,5,9,11,13,17,25,29,30,34,35,36,38,39,42,46,51,54,55,57,58,59,62,64,67,71,72,75],foundat:[17,24,29,54,57,77],founded:[17,24],founifi:2,four:[8,17,25,34,52,54,55,57,71],fourier:[17,24],fourth:[17,54,57],fr:[17,24,25,27,53,75,77],frac:[17,26,31,34,35,38],fraction:[7,11,17,24,27,29,37,57,71],fragil:[17,54,57,59,60,63,66],fragment:[55,57,71],frame:[17,52],framework:[2,17,24],franc:[24,77],francoi:17,frank:[17,77],free:[11,17,24,26,34,44,52,54,55,57,58,62,64,71,75,77],freedom:17,freek:24,freeli:[14,57],freez:13,frege:24,freiburg:77,french:17,frequenc:17,frequent:[11,17,25,53,57,66,67,71],fresh:[3,14,17,24,25,31,34,53,57,58,64,66,67,71],freshid:17,freshnamespac:40,freund:24,frexp:17,frexp_spec:17,frh:5,friendli:[17,24,52],frii:17,fring:17,from:[2,3,4,5,6,8,9,10,11,12,13,14,17,24,25,26,27,28,29,30,31,34,36,37,38,39,40,41,42,43,46,51,52,53,54,57,58,59,60,62,63,64,66,67,71,72,73,75,77],front:[57,59],frozen:24,frshiftexp:27,fs:[2,71],fset:[17,27,60],fsetavl:17,fsetdecid:17,fsetfullavl:17,fsetinterfac:17,fsetproperti:17,fst:[17,24,27,35,42,46,71],fst_list_prod:17,fta:24,ftorradix:8,ftp:77,fubar:57,fulfil:[2,17,67],full:[13,14,17,24,25,30,34,43,46,52,57,58,64,66,71,77],fuller:24,fullfil:17,fullgrammar:71,fulli:[2,3,8,17,24,26,28,31,32,35,38,44,51,52,53,54,55,58,59,64,66,71,72],fun:[2,3,4,5,6,9,10,11,12,13,14,17,25,26,27,29,30,31,32,34,35,37,38,40,41,42,43,44,46,54,55,57,58,59,64,66,67,71,72,75],fun_scop:17,funapp:71,func_scheme_def:72,funclass:[4,17,41,71],functin:17,function_scop:[14,17,25,34,46,57,67],functions_in_zfc:24,functor:[0,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,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],functor_app_annot:35,functori:17,fund:17,fundament:[17,24,31,57],funext_down:14,funext_typ:14,funind:[17,57,59,72],funind_plugin:[57,72],further:[3,17,27,30,35,41,51,52,54,55,57,64,66,67,71],furthermor:[10,17,24,25,26,29,31,33,34,51,52,55,57,63,66],futur:[4,9,10,13,14,17,32,34,41,51,52,53,57,62,66,71,77],fuzz:17,fv:11,g0:[60,67],g1:60,g2:60,g:[3,4,5,9,10,13,14,17,24,27,28,29,30,31,34,35,36,41,43,44,46,52,53,54,55,57,58,59,60,62,64,66,67,71,75,77],g_1:57,g_:57,g_equat:53,g_i:34,g_n:57,ga:77,gabriel:17,gadt:2,gain:[17,24],gallego:17,gallina:[11,17,25,27,41,66,75],gamma:[0,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],gan:17,gap:57,gappa:17,garbag:[17,75],gariano:17,garillot:17,garrigu:17,gather:[17,24,27,55,57,58],gave:[17,24,58],gc:[17,66],gcd:[17,59],gcd_comm:59,gcd_mod:17,gcd_mod_l:17,gcd_mod_r:17,gcd_mul_diag_l:17,gcd_uniqu:17,gcd_unique_alt:17,gcst19:[12,39,77],gdk_use_xft:52,ge:[5,17,27],gear:[8,52],geb:5,geb_g:17,gen:57,gen_constant_modul:17,gen_item:57,gen_x:67,genarg:52,gener:[5,7,8,9,12,13,16,17,24,25,27,28,30,31,32,34,35,36,37,38,39,40,43,46,51,52,53,58,59,60,61,62,64,66,75,77],generalis:57,generaliz:[13,17,44],generalize_eq:67,generalize_eqs_var:67,generalizing_bind:[28,44],generer:17,genericminmax:17,genral:17,geometri:[7,24],geoproof:17,georg:[17,57,77],georgian:29,germani:77,get:[2,5,9,11,13,14,17,24,25,27,28,29,34,36,42,51,52,53,55,58,59,60,64,66,67],get_current_context:17,get_set_oth:36,get_set_sam:36,get_sign:11,gett:37,getter:17,geuver:24,gexpn0:57,gexpn1:57,gexpn_add:57,gfail:[17,54,60],ghc:17,giana:17,gianfranco:77,giarrusso:17,gift:[24,77],gilbert:[17,77],gill:[24,72],gimenez94:[34,77],gimenez95:[30,77],gimenez98:[30,77],gimenezcasteran05:[30,77],gintuit:17,giovini:77,girard:[24,77],gist:17,git:[17,53],github:[2,5,17,51,52,71],gitlab:17,gitter:17,give:[2,3,4,5,7,8,9,11,13,14,17,24,25,26,27,28,29,31,32,34,35,37,40,41,42,45,46,51,52,53,54,55,57,58,59,64,66,67,71,75],give_up:17,given:[2,3,4,5,9,10,11,13,14,17,24,25,27,28,29,32,35,36,37,40,41,42,43,44,46,51,53,54,55,57,58,59,60,62,64,66,67,71,72,74,75],glanc:57,glob:[17,24,51,75],glob_constr:55,glob_term:17,global:[2,3,4,5,9,13,17,24,25,26,28,29,31,32,34,35,37,38,39,41,42,44,51,53,55,57,58,59,60,62,64,66,67,75],globalis:24,globfil:53,glondu:17,gloss:37,glossari:[16,17,25,29],glt89:[66,77],glu:3,gmatch_hyp_pattern:55,gmatch_pattern:55,gmatch_rul:55,gmn:[7,77],gmp:17,gnu:[17,51,53],go:[2,5,9,17,24,30,42,51,52,54,55,57,59,60,64,67,71,75],goal0:[6,43,58,66],goal:[3,6,7,8,9,12,13,14,17,24,25,27,29,31,34,35,36,37,38,42,43,44,52,53,59,60,61,62,64,71,72,74],goal_match_list:55,goal_occurr:58,goal_pattern:54,goal_selector:54,goal_tact:54,goe:[17,53,55,59,66],goir:77,gone:17,gonthier:[17,57,77],good:[11,17,53,54,55,57,66],googl:[51,53],got:[17,34,67],gothenburg:77,gothic:29,gotten:52,goubault:24,govern:[17,41,44,52,67],gr:77,grab:17,gradual:[17,58],grai:[29,52],grain:[2,17,41],grammar:[10,17,25,28,29,54,55,57,58,62,71],grant:17,granular:[52,55],graph:[2,14,17,24,25,39,54,72],graphic:[17,25,29,51,52],graphviz:[14,17],grasp:57,grate:17,grayson:17,great:[31,64],greater:[14,17,24,34,52,71],greatli:[17,24],greek:[17,29,75],green:[17,29,52,66],greg:17,gregersen:17,gregoirel02:[64,77],gregori:17,grep:59,grinberg:17,groebner:17,groot:77,gross:17,ground:[14,17,54,62,71,75],group:[2,4,17,24,37,42,52,53,54,57,58,60],grow:[24,54,55,59],growth:54,gruetter:17,gruin:17,grundlagen:24,gt:[17,27,42],gt_wf_rec:2,gt_wf_rect:17,gtb:5,gtb_gt:17,gtk2:17,gtk3:17,gtk:[17,52],gtk_accel_path:52,gtk_csd:17,gtk_theme:52,gtksourceview:[17,52],guarante:[4,14,17,51,52,53,55],guard:[17,24,25,27,30,32,34,41,44,46,57,59,64,66,67,71,72,77],guarded:[9,66],guess:[2,4,11,17,32,43,53,57,67],gui:[24,52,76],guid:24,guidelin:17,guillaum:17,gulp:66,gv:[14,17],gwhy:17,gyesik:77,gz:[17,51,53],gzip:53,gznd11:[42,77],h0:[54,55,57,58,62,64,66,67],h1:[11,17,34,43,54,55,57,58,62,66,67],h23:57,h2:[17,34,43,54,55,57,58,67],h2_0:67,h2_:67,h3:[58,67],h:[3,4,6,9,11,12,13,14,17,24,27,34,40,44,46,51,54,55,57,58,62,64,66,67,72,75,77],ha:[2,3,4,5,6,8,9,11,12,13,14,17,24,25,26,27,28,29,30,31,32,34,35,36,37,38,39,40,41,42,43,44,46,51,52,53,54,55,57,58,59,60,62,63,64,66,67,71,72,73,74],haan:17,haani:17,had:[9,13,17,24,42,53,54,55,66],hal:77,half:[17,24,37,66],hallberg:17,hand:[3,10,12,13,17,25,27,29,33,35,52,53,54,55,57,58,64,67,71,72],handi:[17,71],handl:[2,3,8,9,11,17,24,26,37,43,46,53,55,57,58,59,61,62,66,67,71],hangul:29,hao:17,happen:[2,4,9,10,13,17,34,38,46,52,54,55,57,58,64,71,72],hard:[17,55,59,64],hardcod:17,harder:[4,17,58],hardwar:[2,8,24],harm:34,harmless:[34,51],harrison:5,harsh:17,harvei:17,has_evar:17,hash:17,haskel:[2,13,17,24,25,57,64,77],hasn:35,have:[2,3,4,5,7,8,9,10,11,12,13,14,17,24,25,26,27,28,29,30,31,32,33,34,35,36,37,39,40,41,42,43,44,46,51,52,53,55,58,59,60,62,64,66,67,71,73,75],haven:[52,54],hayashi:24,hb:[57,58],hd:[17,30,34,57,72],hd_error_skipn:17,he:[11,17,24,57],head:[3,10,13,14,17,24,26,27,30,35,41,42,44,53,54,55,57,58,59,60,64,67,71],headconcl:[17,59],header:[17,51,75],headhyp:[17,59],heap:[17,54,66],heap_word:66,heapsort:[17,24,27],heart:33,heavi:2,heavili:17,hebb:17,hebrew:[17,29],heel:54,heidelberg:77,heiko:17,held:24,helg:17,helm:[17,24],help:[2,3,8,13,14,15,16,17,24,25,27,29,41,46,51,52,53,54,55,57,58,60,62,67,75],helper:[25,59],henc:[2,3,4,5,8,9,13,14,17,26,34,37,42,51,53,54,57,58,64,67,71],hendrik:17,henk:24,henri:[17,24],heq:[17,54,67],heq_n0:9,heq_n:9,heql:67,heqp:67,her:24,herbelin:[17,24,46],here:[2,3,4,5,9,11,13,14,16,17,24,27,29,31,33,34,35,37,38,41,42,44,46,51,52,53,54,55,57,58,59,60,64,66,67,71,75],hereaft:[26,30,55,57],herm:17,herman:24,heterogen:[17,67],heurist:[2,5,14,17,55,57,58,66],hex:17,hex_int_scop:71,hex_n_scop:17,hex_nat_scop:71,hex_positive_scop:17,hex_uint_scop:71,hex_z_scop:17,hexa:71,hexadecim:[17,27,29,36,52,59],hexdigit:29,hexnat:29,hf:[34,51],hfg:57,hget_evar:17,hi:[17,24,34],hid:17,hidden:[17,24,25,27,53,57,71,75],hidden_arrow:12,hide:[17,25,34,41,44,57,58,66,71],hierarch:[24,35],hierarchi:[14,17,24,25,34,39,51],high:[14,17,24,25,35,59,60,66,72],higher:[3,14,17,24,25,27,40,51,54,57,58,59,60,64,67,71,73,77],highest:71,highli:[10,43,60,63],highlight:[17,51,52,53,57,63,66],higman:2,hijack:17,hilbert:[5,7,17],hinder:17,hindlei:[55,77],hindranc:54,hint:[3,13,14,17,24,25,27,35,38,54,62,64,75],hint_info:[13,60],hintbas:[55,60],hintdb:[13,17,55,60],hints_regexp:60,hiragana:29,histor:[17,25,44,55],histori:[17,25,26,53,59,66],hivert:17,hl:67,hloc:58,hlt:27,hn:66,hnat:44,hnf:[17,24,41,42,57,58,64,67],hnm:57,ho:[17,29,58],hoc:[2,3,17,71,77],hoist:17,hol:5,hold:[3,4,17,30,34,35,40,42,55,58,75],hole:[9,13,17,24,25,40,43,46,55,57,58,59,62,66,67,71],holland:77,home:[17,51,52,53],homebrew:17,homogen:[3,17],homotopi:17,honor:[2,17,51,57,71],honour:57,hood:[5,17],hook:[17,53],hope:[24,52],hopefulli:[17,55],horizont:[17,29,53,71,75],horror:25,host:17,hott:[17,40],how80:[26,66,77],how:[2,7,8,13,17,24,25,27,29,30,34,35,37,42,43,45,51,53,54,57,58,59,60,62,64,67,71,72,74,77],howard:[24,26,66,77],howev:[3,4,5,9,12,13,14,17,24,27,29,34,36,37,41,43,44,46,51,52,53,54,55,57,58,64,66,67,71,72],hp:[57,67],hpa:57,hpb:57,hq:[57,67],hqa:57,hqab:57,hrec:57,hresolve_cor:17,hspace:[26,31,34,35,38],html:[17,25,29,53],http:[2,5,17,24,25,27,50,51,52,53,59,64,71,75,77],hue88:[24,77],hue89:[24,66,77],huet:[24,77],hug:17,huge:[8,11,17,54,57,66],hugo:[17,24,46],hugunin:17,human:[17,25,58,75],hundr:[11,64],hur:17,hv:71,hx:[12,57,58],hy:58,hybrid:17,hydra:2,hyp0:57,hyp:[17,24,55,57,59,66,71],hyp_occ:58,hyp_valu:17,hyperlink:[17,25,29],hypertextu:24,hyphen:74,hypid:58,hypothes:[3,5,9,13,17,24,25,28,32,34,51,57,60,62,64,67,71],hypothesi:[3,9,11,17,24,25,27,28,29,34,38,55,57,59,60,62,64,66,67,71,72,75],hz:54,i1:[34,71],i2:71,i:[0,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],i_1:[7,11,34,35],i_2:[11,57],i_:[3,34,57],i_block:57,i_i:35,i_ind:[46,71],i_item:57,i_j:[34,35],i_k:[7,34,35],i_l:34,i_n:[11,57],i_not_i:34,i_p:34,i_pattern:57,i_rec:[46,71],i_rect:[46,71],i_sind:[46,71],i_view:57,ia:17,icfp:77,icon:[17,52],id0:14,id1:17,id:[3,4,9,10,14,17,24,26,34,35,42,44,51,52,53,54,55,57,58,64,66,71,75],id_1:17,id_fct_funclass:4,id_n:17,id_rew:10,id_str:71,iddec:53,idea:[11,17,34,42,54],ideal:7,idem:24,ident0:51,ident1:51,ident:[2,3,5,6,9,10,11,12,13,14,17,24,25,27,28,29,30,31,32,34,35,37,38,40,43,44,46,51,53,55,57,58,59,60,62,64,66,67,71,72,73,74],ident__i:6,ident_decl:[4,9,13,28,30,32,34,37,38,40,42,59],ident_or_anti:55,identifi:[2,3,9,14,17,24,25,28,29,30,31,35,38,40,41,43,44,46,51,52,53,54,55,57,58,60,66,67,72,75],identityt:17,ideograph:29,idiom:[17,54,55,57,66],idl:52,idn:17,idp:57,idtac:[14,17,25,52,55,57,60,66,71,74],idx:57,ieee:[17,36,77],iempti:71,if_then_els:[17,71],ifeq:53,iff:[3,17,26,27,31,57,59,71],iff_reflex:59,iff_symmetr:59,iff_tran:17,ifflr:57,iffrl:57,ifft:17,ifi:17,igler:17,ignat:17,ignor:[4,13,14,17,24,27,29,31,34,35,44,51,52,53,54,57,58,60,64,66,71],ih:67,ihl:67,ihm:57,ihn0:[67,72],ihn:[57,66,67],ihp:67,ihterm:67,ihu:57,ihv:57,ik:17,ikebuchi:17,ikfprintf:17,ill:[2,4,9,10,17,24,30,34,51,55,64,71,72],illeg:4,illtypedinst:17,illustr:[5,17,34,46,57,60,64],imag:[3,11,17,24,51,52,66],imai:17,imedi:60,immedi:[17,24,27,54,55,57,58,59,60,66],immediatli:17,immut:36,impact:[2,17,53,66,71],imped:54,imper:[17,24,55],impl:[3,5,59],impl_reflex:59,implb:[5,17,27],implb_andb_distrib_r:17,implb_contraposit:17,implb_curri:17,implb_false_iff:17,implb_false_l:17,implb_false_r:17,implb_negb:17,implb_orb_distrib_l:17,implb_orb_distrib_r:17,implb_sam:17,implb_true_iff:17,implb_true_l:17,implb_true_r:17,implement:[3,8,11,12,13,17,24,25,27,29,34,35,36,37,39,43,46,54,55,57,58,59,60,62,64,66,67,71,72,77],implementor:59,impli:[2,3,10,14,17,24,30,34,57,67,71],implic:[3,17,26,27,28,42,54,57,60,66,67,71],implicit:[2,3,5,9,13,17,24,25,28,33,34,37,38,42,43,45,51,53,55,57,58,59,66,67,75],implicit_bind:[28,44],implicitli:[3,13,14,17,24,34,51,55,60,64],implict:41,implypp:17,import_categori:[17,35,59],importantli:17,impos:[24,30,34,57],imposs:[5,17,34,46,53,58,67],impract:53,impred:[2,12,14,17,24,25,34,51,53,77],improp:17,improv:[2,3,8,11,17,24,29,52,54,57,67],inE:17,in_concat:17,in_cons_iff:17,in_context:17,in_dec:17,in_elt:17,in_elt_inv:17,in_flat_map_exist:17,in_goal:17,in_hd:67,in_hyp_a:58,in_iff_nth_error:17,in_in_remov:17,in_inj_comp:17,in_left:17,in_nth:17,in_remov:17,in_rev:17,in_right:17,in_shiftin:17,in_tl:67,inabl:64,inaccess:17,inact:66,inadvert:[17,52],inc:17,incant:57,incident:17,incl:[17,59],incl_app_app:17,incl_app_inv:17,incl_cons_inv:17,incl_exist:17,incl_filt:17,incl_foral:17,incl_forall_in_iff:17,incl_l_nil:17,incl_map:17,incl_nil_l:17,incl_refl:59,inclass:17,includ:[2,3,5,8,9,12,13,14,17,24,25,27,28,29,34,35,36,38,39,40,41,43,44,51,52,53,54,55,57,59,60,62,64,66,67,71,73,75],include_subdir:53,inclus:[14,17,54,55],incoher:[17,46],incom:[4,17],incompar:71,incompat:[14,24,25,34,41,46,57,59,66,71],incompatibili:17,incompatibilit:24,incomplet:[5,8,10,17,24,46,58,66,67,71],inconsist:[2,8,10,12,14,17,24,26,34,39,44,51,59,66,67,71],incorrect:[2,8,12,14,17,25,34,37,46,52,57,66],incorrectli:[12,17,55],incr_fct:4,increas:[3,5,8,17,24,53,57,62],incred:55,increment:[17,24,30,31,32,33,34,38,55,66],incur:[17,66],ind1:35,ind2:35,ind:[0,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],ind_bool:59,indag:77,inde:[3,4,11,12,13,14,17,25,26,29,30,34,35,40,41,42,43,44,46,53,54,55,57,58,60,64,66,67,71,72],indefclass:17,indefinit:17,indefinitedescript:17,indent:[8,17,25,66,71,75],independ:[2,13,14,17,24,34,51,52,53,54,55,57,67],indetermin:57,index:[3,13,17,24,25,26,27,29,39,40,44,52,58,60,64,66,67,73,75],index_iota:57,indic:[2,8,11,12,13,14,17,24,26,31,34,35,39,40,41,42,43,46,51,52,53,54,57,58,59,62,64,66,67,71],indirect:[17,64],indirectli:[17,24,58,59,60,74],indistinguish:[14,37],individu:[17,53,55,64,67,71],indp1:35,indp2:35,indp:[0,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],indpstr:[0,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],indrec:17,induc:[17,24],induct:[4,5,9,10,11,12,13,14,17,24,25,27,29,30,31,32,33,35,37,41,42,44,52,54,55,57,58,59,60,62,64,65,66,73,75,77],induction_arg:[55,67],induction_claus:[55,67],induction_ltof1:17,induction_ltof2:2,induction_principl:67,induction_test2:67,induction_test:67,inductive_definit:[30,34],ineffici:[5,17,24,57],inequ:[5,17,24,60],inexact:27,infam:17,infer:[3,4,9,10,13,14,24,25,26,34,37,40,41,42,45,46,51,57,58,60,62,67,71],infin:[27,30,71],infinit:[12,27,30,34,39],infinite_loop:34,infix:[2,14,17,24,25,27,42,57,58,64,74],inflat:17,influenc:[17,24,34],info:[5,17,54,60],info_auto:[17,60],info_eauto:[17,60],info_trivi:17,infoh:54,inform:[2,3,4,10,12,13,14,17,24,25,26,27,29,30,34,37,39,41,42,43,44,46,51,52,53,54,55,57,58,59,60,62,64,67,72,75,77],informatiqu:[24,77],infrastructur:[3,25,42,53],ing:[17,74],ingredi:54,inhabit:[14,29,31,32,34,37,40,43,46,51],inher:57,inherit:[17,24,25,42,52,55],inhibit:[17,57],ini:52,init:[9,14,17,27,28,35,51,54,55,58,59,60,66,67,71],initi:[2,6,7,11,13,17,24,27,29,38,46,52,53,54,55,57,58,59,60,62,63,64,66,67,71,74,75],initialr:11,inj:62,inj_compr:17,inj_land:17,inj_ldiff:17,inj_lor:17,inj_lt:57,inj_lxor:17,inj_shiftl:17,inj_shiftr:17,inject:[0,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],inject_nat:17,injective_map_nodup_in:17,injtyp:[5,17],inl:[27,40,57],inleft:27,inlin:[17,24,25,28,35,64,66,72,75],inner:[2,14,17,35,42,43,54,55,57,59,62,64,66,67,71,75],innermost:[54,71],input:[3,4,9,10,14,17,25,27,29,35,44,46,51,54,57,58,60,64,71,72,74,75],inputenc:75,inr:[17,27,40],inr_0:17,inr_1:17,inr_archim:17,inr_izr_inz:17,inr_unbound:17,inria:[17,24,25,27,53,75,77],inright:27,ins:[17,58,59],insarov:17,insensit:17,inser_trans_r:17,insert:[3,4,9,12,13,17,24,25,29,41,46,52,53,55,57,66,71,75],insid:[2,3,4,8,9,13,14,17,24,25,28,29,34,35,38,46,52,55,57,58,59,60,64,66,67,71,74],insofar:55,inspect:[2,17,57,59],inspir:[17,24,75],inst:37,instabl:17,instal:[17,25,27,35,51,52,64,66,72,73],installcoqdocroot:17,instanc:[2,3,4,5,10,11,12,14,17,25,26,27,28,29,30,31,34,35,36,37,38,39,40,41,42,44,46,51,52,53,55,57,58,59,60,62,64,66,67,71,75],instancenam:13,instanti:[3,10,13,14,17,24,34,35,43,44,54,55,57,58,60,62,67,71],instantiate_ltac_vari:58,instantli:57,instat:42,instead:[2,3,4,7,8,11,12,13,14,17,24,26,28,33,34,35,36,37,43,44,46,51,52,53,54,55,57,58,59,60,62,64,66,67,71,72,74,75],institut:[24,27],instruct:[2,5,17,53,58,59],instrument:61,insub:57,insubt:57,insuffici:[14,17,51],insur:24,int31:17,int63:[17,71],int63_eq:[36,59],int63_typ:[36,59],int63not:17,int_mult:57,int_of_nat:2,int_or_var:[3,54,66,71],int_part_frac_part_spec:17,int_part_spec:17,int_scop:17,int_wrap:71,int_wrapp:71,intead:17,integ:[2,3,7,11,14,17,24,25,29,34,39,52,53,54,55,57,59,60,64,66],integr:[10,11,17,24,25,27,51,52,57,61,73],intellig:[24,42],intend:[3,17,24,28,32,39,51,57,64,66,71],intens:[11,17,24,64],intent:[17,24,28,57],intention:51,intepret:17,inter:[24,53],interact:[3,10,13,17,24,25,32,33,37,38,40,42,43,52,59,65,66,67,75,76,77],interchang:[53,66],interdepend:25,interest:[2,4,5,11,17,24,31,42,54,57,67],interfac:[2,17,24,25,35,52,53,66,74,75,76],interfer:[57,71],interleav:[11,17,58],intermedi:[17,27,57,66],intermediari:[2,64],intern:[3,5,11,14,17,24,25,31,34,37,44,51,53,54,55,58,60,62,66,67,71,72,73,74,77],internal_:59,internet:52,internship:24,interpet:58,interpol:[17,53,75],interpret:[3,5,9,11,13,17,24,25,27,29,32,34,35,41,44,51,52,53,54,55,59,75],interrupt:[17,52,54,59],intersect:9,intertwin:[17,57],interv:52,intervent:52,intf:17,intmap:[17,24],intric:[54,55],intro:[3,5,11,12,13,17,24,25,27,34,42,43,44,52,54,55,60,62,64,66,67,71,72],introa:34,introduc:[3,5,8,10,11,13,14,17,24,25,28,30,31,34,35,37,38,43,44,46,51,52,55,57,58,59,60,62,66,67,71,72,75],introduct:[7,13,17,24,30,34,62,67,71],introl:58,intron:57,intronf:57,introntf:57,intropattern:[17,55,58,67],intror:58,intros_until:55,intuit:[4,11,17,24,29,55,58,62],intuition_solv:[17,62],intuitionist:[17,24,25,27,34,57,62,77],intuitionnist:77,inv_high:14,inv_low:14,invalid:[17,24,40,52,54,59,64,66,71],invalid_argu:[17,55],invari:[14,17,55],invariant_ind:14,invariant_rec:14,invariant_rect:14,invariant_sind:14,invers:[3,11,17,24,25,27,31,58,60,64,72,77],inverse_imag:17,inversion_clear:67,inversion_sigma:17,invert:[13,17,57,67,72],invert_con:67,investig:[17,24,77],invis:[17,53,57],invit:[24,42],invoc:[25,53,54,57,59],invok:[11,17,34,51,53,59,60,66,67,75],involv:[3,4,9,12,17,24,25,26,34,41,42,51,52,53,54,57,59,60,62,64,67],inz:17,io:[17,25],iota:[0,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],ip_i:34,ipat:[17,57],ipattern:17,ipr_2_xh:17,ipr_2_xi:17,ipr_2_xo:17,ipr_eq:17,ipr_ge_1:17,ipr_gt_0:17,ipr_ipr_2:17,ipr_l:17,ipr_lt:17,ipr_not_1:17,ipr_xh:17,ipr_xi:17,ipr_xo:17,irif:77,irr_high:14,irr_low:14,irreduc:[17,37,64,71],irrefut:[17,25,32,40,57],irrelev:[14,17,25,32,33,34,39,54,55,57,64,77],irrelevant_ind:14,irrelevant_rec:14,irrelevant_rect:14,irrelevant_sind:14,irrevers:[17,24,64],irst:77,is_arrai:17,is_clos:17,is_conj:54,is_const:17,is_constructor:17,is_disj:54,is_double_moins_un:17,is_empti:17,is_evar:[17,54],is_float:17,is_ind:[17,54],is_law:42,is_law_:42,is_proj:17,is_tru:[12,57],is_true_eq_tru:12,is_uint63:17,is_zero:46,isaac:17,isbn:77,island:77,islezero:17,isn:[9,10,17,28,52,57,58,60,64,66,67],iso:[17,75],iso_axiom:54,isol:57,isomorph:[24,25,46,55,62,66,67,77],isprop:5,isquash:12,isquash_sind:12,issac:77,issu:[2,3,24,25,46,52,54,55,58,64,66,71,73],issucc:27,isum:71,iszero:17,ital:[29,53,66,75],italic:[17,75],itarget:17,item:[17,24,25,29,52,54,55,58,60,64,66,67,71,75],iter:[3,5,13,17,25,26,27,28,30,71],iter_add:17,iter_ind:17,iter_invari:17,iter_nat:17,iter_op:17,iter_op_correct:17,iter_rect:17,iter_succ:17,iter_succ_r:17,iter_swap:17,iter_swap_gen:17,ith:46,ito:77,itp:[17,77],its:[2,3,4,5,6,9,10,11,12,13,14,17,24,25,27,28,29,30,31,32,34,35,36,37,38,42,43,44,46,51,52,53,54,55,57,58,59,60,62,63,64,66,67,71,72,73,74,75,77],itself:[2,3,8,9,11,12,13,14,17,30,34,39,40,41,42,43,44,51,53,54,55,57,58,60,63,64,67,71],itzhaki:17,iunit:71,izr:[5,17,71],izr_neq:17,izr_pos_xi:17,izr_pos_xo:17,j:[5,6,8,14,17,24,25,26,34,36,39,43,51,54,57,64,72,77],jablonka:17,jacek:[17,24],jacob:17,jacqu:17,jai:17,jaim:17,jame:17,jan:[17,24,77],januari:[17,24,77],jason:17,jasongross:17,jasper:17,javadoc:75,jean:[2,17,24,77],jedit:17,jef:53,jerri:17,jesper:[17,77],jesu:17,jfehrl:52,jim:17,jm:24,jmeq:[17,67],jmeq_eq_dep:17,joachim:17,job:[8,52,53,54,57],johann:17,john:[5,77],join:[5,24],joint:24,jonathan:17,jone:77,jose:17,jouannaud:77,jourdan:17,journal:77,jouvelot:17,jp:17,jr:17,json:[2,17,51,53,59],juan:17,judg:54,judgement:24,judgment:[26,35,59,77],juli:[17,24],julien:[17,72],julin:17,jump:[8,17,52,57],june:[17,24],jung:17,jurgensen:17,jussieu:17,just:[2,3,4,8,9,11,13,17,24,28,31,34,35,37,41,42,46,51,52,53,55,57,58,59,60,62,64,66,67,71,75],justif:27,justifi:[17,27],jut:24,k1:57,k2:57,k:[2,3,6,14,17,24,26,34,42,54,57,67,72,77],k_1:34,k_i:34,k_j:34,k_n:34,kaiser:17,kaliszyk:17,kalla:17,kamil:17,karl:17,karolin:17,karolina:17,karpiel:17,kartik:17,katakana:29,kate:17,kayla:17,kazuhiko:17,keep:[2,12,14,17,24,33,34,36,42,46,52,53,55,57,64,67],keeper:17,keepsingleton:[2,17],kei:[17,25,41,42,55,57,59,64,66,71],keller:17,kenji:17,kent:77,kept:[14,17,24,36,53,67,75],kernel:[8,9,10,12,24,25,27,29,32,33,36,37,38,41,45,46,53,55,58,59,64,66],ketonen:24,keyboard:[52,59],keystrok:52,keyword:[17,24,25,28,29,32,37,40,46,55,57,64,71,75],khalid:17,khanh:17,kil:17,kill:17,kind:[2,8,10,11,17,25,27,29,34,42,46,53,55,57,59,67,72],kit:17,klausner:17,kleen:[24,60],kloo:17,knaster:24,know:[2,8,17,24,27,32,34,42,46,52,53,54,55,57,59,60,62,64,67,71],knowledg:[17,25,71],known:[2,8,10,12,13,17,24,27,30,33,34,39,41,44,51,55,57,66,71],knownfil:53,knowntarget:53,ko:53,konstantino:17,kosogorov:17,krebber:17,krivin:[17,64],kuefner:17,kunz:17,kuper:17,kw:[0,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],kwend:[0,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],kyoto:24,l0:[46,54,64],l1:[42,54],l1_tactic:54,l2:[42,54],l2_tactic:54,l2r:17,l3_tactic:[54,66],l:[0,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],l_inj:17,l_r_neq:17,la:[13,17,24,52,55,77],lab:24,label:[2,8,14,17,29,54,59],lablgtk2:17,lablgtk3:17,laboratori:24,lack:[17,53,54,57],lafont:[17,77],lam:[26,34],lambda:[2,3,10,11,17,31,52,55,64,67,71,77],lambo:24,lampropoulo:17,land:[5,17,59,71],land_comm:59,land_even_even:17,land_even_l:17,land_even_odd:17,land_even_r:17,land_le_l:17,land_le_r:17,land_odd_even:17,land_odd_l:17,land_odd_odd:17,land_odd_r:17,land_on:59,landau:24,landmark:17,lang:77,langl:17,langston:17,languag:[3,9,11,14,26,29,36,37,39,40,41,46,53,54,63,64,65,66,74,75,77],lannion:24,laport:17,lappli:58,lar:17,larchei:17,larg:[11,14,17,25,26,29,34,35,39,52,53,54,57,61,64,66,67,71,75],larger:[2,13,14,17,25,51,52,57,60,71,75],largest:[57,71],larri:[17,24],lass:[17,77],lasson:17,last:[4,5,9,17,24,32,34,35,37,38,42,46,51,52,53,54,55,57,58,59,60,64,65,66,67,71,72],last_ind_list:57,last_last:17,last_length:17,last_spec:57,last_spec_ind:57,last_spec_rec:57,last_spec_rect:57,last_spec_sind:57,lastadd:57,lastcas:57,lastli:75,lastp:57,lastseq0:57,late:[8,17,24,25,64],later:[11,17,25,31,32,43,44,50,53,55,57,58,66,67,71],latest:[17,25,50],latex:[0,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,54,55,56,57,58,59,60,61,62,63,64,65,66,67,68,69,70,71,72,73,74,76,77],latin1:75,latin:[17,29],latter:[3,11,17,28,34,35,42,51,54,55,57,58,64,66,67,75],lattic:4,launch:[2,13,17,25,52,53],laurenc:[17,57],laurent:[11,17,24],law:[17,24,25],lax:[17,55,60],layer:[10,17,25],layout:17,lazi:[2,8,9,12,17,24,55,64],lazili:[8,17,30,54],lazy_and:17,lazy_goal_match0:17,lazy_impl:17,lazy_or:17,lazymatch:17,lb:13,lbase:17,lceil:5,lcf:[24,55],lcm0:17,lcm:[17,59],lcm_comm:59,ldexp:17,ldexp_spec:17,ldiff:59,ldiff_even_even:17,ldiff_even_l:17,ldiff_even_odd:17,ldiff_even_r:17,ldiff_le_l:17,ldiff_odd_even:17,ldiff_odd_l:17,ldiff_odd_odd:17,ldiff_odd_r:17,ldot:[3,7,34],ldshiftexp:27,le0:42,le:[3,5,13,14,17,24,27,42,46,52,55,57,64,67,77],le_:27,le_add_l:17,le_class:42,le_div2:17,le_div2_diag_l:17,le_epsilon:17,le_eqb:13,le_gt_dec:[2,57],le_ind:[27,46,67],le_ipr:17,le_lt_dec:[2,17,24],le_lt_tran:43,le_m_n:57,le_minu:[17,72],le_n:[27,57,67],le_n_m:57,le_n_p:57,le_not_lt:17,le_plus_r:17,le_rec:67,le_rect:67,le_sind:[27,46,67],le_tran:58,lead:[2,10,14,17,24,26,29,34,39,57,58,60,64,71,74,75],leaf:[34,67],leak:17,learn:[2,17,25,54,72],least:[2,3,12,13,17,25,28,29,30,34,41,46,52,53,57,58,64,66,67,71,72,74,75],leav:[12,13,17,32,35,52,54,57,58,59,60,64,66,67],leb:[5,9,17,27,57,59],leb_implb:17,lectur:77,led:[17,24],ledinot:24,lee:[17,77],lef:46,lefanu:17,left:[0,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,68,69,70,71,72,73,74,75,76,77],lefta:71,leftarrow_:11,leftmost:[17,34,41,58],legaci:[2,3,5,6,9,11,14,17,27,29,34,36,40,42,43,51,54,55,57,58,59,60,64,66,71,72],legacy_attr:[9,14,29,35,40],legal:[17,31,34],legibl:57,legitim:24,lego:24,leibniz:[3,5,7,11,13,17,24,25,27,35,40,57,58,67],leivent:17,lel:59,lel_refl:59,lele_eq:42,leminv:67,lemm:24,lemma:[3,5,11,13,14,17,24,25,32,34,35,36,38,42,44,46,54,57,58,59,60,62,64,67,72],lemmata:17,len:54,lenght:27,length:[0,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],length_app:17,length_combin:17,length_con:17,length_concat:17,length_firstn:17,length_flat_map:17,length_fst_split:17,length_list_pow:17,length_map:17,length_nil:17,length_prod:17,length_rev:17,length_seq:17,length_skipn:17,length_snd_split:17,length_tl:17,length_to_list:17,length_zero_iff_nil:58,lennart:17,lennon:17,leo:[46,67],leonida:17,lepigr:17,leq:[34,42,57],leq_add_sub:57,leqn:57,ler90:[64,77],lerai:17,leroi:[17,24,77],lescuy:17,less:[2,4,8,11,14,17,24,34,46,51,53,54,55,57,59,60,64,71,77],let02:[2,77],let:[0,1,2,3,4,5,6,7,8,9,10,11,12,13,14,15,16,17,18,19,20,21,22,23,25,26,27,28,29,30,31,33,34,35,36,37,38,39,40,41,42,43,44,45,47,48,49,50,51,52,53,55,56,58,59,60,61,62,63,64,65,66,67,68,69,70,71,72,73,74,75,76,77],let_claus:54,letan:17,letin:[0,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],letouzei:[2,17,24,77],lettac:24,letter:[17,24,26,27,29,37,46,51,55,71,75],level:[8,13,14,17,24,25,26,27,31,35,36,37,41,42,46,51,52,53,54,57,59,64,66,67,71,72,73,75],lewycki:17,lex:75,lexer:66,lexic:[2,17,25,51,59,71,75],lexicograph:[7,11,53],lexicographic_exponenti:17,lexicographic_product:17,lfloor:5,lgth:34,lh:[55,57,59],li:17,lia:[17,25,54,55,57,60],lia_ltac1:55,lib:[17,24,51,53,55,59,75],libc:17,librari:[2,5,8,25,29,35,36,40,41,52,54,57,58,64,66,72,75],lic:77,licens:[25,50],licit:25,lid:57,lident:55,life:17,lift:[3,12,14,17],liftn:17,light:[5,17,24,52,66,75],lighter:[8,13],lightweight:17,like:[2,4,8,9,10,11,13,14,17,24,26,27,29,32,34,35,38,39,41,42,43,46,51,52,53,54,55,57,58,59,60,62,64,66,67,71,72,73,75],likewis:[9,17,55],limit:[3,5,8,9,10,13,14,17,24,27,29,35,41,46,51,52,53,54,55,57,58,59,60,63,64,66,71,72],lincon:5,line:[2,8,10,12,14,24,25,29,42,52,53,54,55,57,58,59,64,66,71],lineag:55,linear:[2,3,11,14,17,24,25,46,51,54,55,57,64],linearintuit:24,liner:[17,25],link:[2,16,17,24,27,46,51,53,57,72,75],linker:[2,24],lint:[17,53],linter:[17,51],linux:[17,35,51,52,53,59,64],lionel:17,lip:[24,77],lirmm:77,lisp:24,list0:[55,71],list1:[55,71],list2:34,list2_ind:34,list2_rec:34,list2_rect:34,list2_sind:34,list3:34,list3_ind:34,list3_rec:34,list3_rect:34,list3_sind:34,list:[0,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,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,56,57,58,59,60,61,62,63,64,65,66,67,68,69,70,71,72,73,74,76,77],list_equiv:3,list_ext:17,list_extens:17,list_ind:[14,34,41,44,46,57,67],list_max:17,list_max_app:17,list_max_l:17,list_max_lt:17,list_power_length:17,list_prod_as_flat_map:17,list_rec:[14,34,41,44,46,57,67],list_rect:[14,34,41,44,46,57,67],list_scop:[17,27,64,71],list_sind:[14,34,41,44,46,57,67],list_sum:17,list_sum_app:17,listdec:17,listing_decidable_eq:17,listn:46,listn_ind:46,listn_rec:46,listn_rect:46,listn_sind:46,listnot:[17,54,72],listset:17,listw:34,liter:[2,5,17,29,36,42,54,55,57,71],literatur:[13,34],littl:[8,9,11,14,17,35,57,64],live:[14,17,51,55],live_word:66,ljt:[54,62],ll1:71,ll:[13,17,34,52,53],llm3:24,ln:17,ln_exists1:17,lnc:77,lnot:[17,75],load:[2,3,5,6,7,9,11,17,24,25,27,29,34,35,36,42,43,54,55,57,58,60,64,66,67,71,72,73],loadabl:17,loadfil:59,loadpath:[17,24,51,53,59],local:[2,3,4,5,9,13,17,24,25,26,28,30,31,32,34,41,42,52,55,59,62,64,66,67,75],localis:24,locallysorted_sort:17,locat:[2,17,24,25,35,51,52,53,54,55],lock:[17,25],lockwood:24,log2:[17,59],log2_it:59,log:[17,24,53,54],logarithm:17,logic:[2,3,9,12,13,14,17,24,25,26,28,29,30,34,35,39,51,57,58,59,61,66,67,75,77],logic_typ:[17,27],logical_dir:24,logical_kind:59,logiqu:77,loic:24,loiseleur:[11,24],lone:[17,71],longer:[3,9,17,24,31,34,38,44,52,53,58,66,67,71],longest:[17,29,34,41,42,57,71,75],longrightarrow:[0,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],look:[4,8,9,11,13,14,16,17,25,51,53,54,55,57,58,59,60,66,67,71,72,75],lookup:11,loop:[17,24,25,53,55,58,60,63],loos:[17,60],lopez:17,lor:[17,59],lor_comm:59,lorenzo:77,lose:[34,67,71],loss:[17,57],lost:[17,30,44,57,67],lot:[3,11,17,24,52,55],lotfi:17,lott:17,louis:17,low:[14,17,25],lower:[14,17,25,52,54,55,57,60,64,71],lowercas:[17,29,37,46,52,55],lowest:[37,54],lpar:77,lqa:5,lra:[0,1,2,3,4,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],lri:[17,24,77],ls:[17,51,53],ls_color:51,ls_l:17,lsl:17,lsp:[17,29,74],lsr:17,lt:[3,9,13,17,27,42,57,71,72],lt_1_ipr:17,lt_1_r:67,lt_div2:17,lt_div2_diag_l:17,lt_eq_lt_dec:17,lt_ipr:17,lt_irrefl:[43,58],lt_mult_left:17,lt_n_m:57,lt_not_l:17,lt_tran:[43,57],lt_wf_double_rect:17,lt_wf_rec:[2,24],lt_wf_rect1:17,lt_wf_rect:17,ltac1:[17,25],ltac1_expr_in_env:55,ltac1val:55,ltac2:[25,35,38,52,53,54,59,63,66,71,74],ltac2_as_ipat:55,ltac2_as_nam:55,ltac2_as_or_and_ipat:55,ltac2_atom:55,ltac2_bind:55,ltac2_branch:55,ltac2_by_tact:55,ltac2_claus:55,ltac2_concl_occ:55,ltac2_constr_with_bind:55,ltac2_convers:55,ltac2_delta_reduct:[17,55],ltac2_destruction_arg:55,ltac2_eqn_ipat:55,ltac2_equality_intropattern:55,ltac2_expr0:55,ltac2_expr1:55,ltac2_expr2:55,ltac2_expr3:55,ltac2_expr5:55,ltac2_expr:[55,71],ltac2_for_each_go:55,ltac2_goal_tact:55,ltac2_hypid:55,ltac2_hypident_occ:55,ltac2_in_claus:55,ltac2_induction_claus:55,ltac2_intropattern:55,ltac2_let_claus:55,ltac2_ltac1_plugin:55,ltac2_match_kei:55,ltac2_match_list:55,ltac2_match_pattern:55,ltac2_match_rul:55,ltac2_naming_intropattern:55,ltac2_occ:55,ltac2_occs_num:55,ltac2_or_and_intropattern:55,ltac2_oriented_rewrit:55,ltac2_plugin:55,ltac2_quot:[17,55],ltac2_red_flag:55,ltac2_reduct:55,ltac2_rewrit:55,ltac2_scop:[55,74],ltac2_simple_bind:55,ltac2_simple_intropattern:55,ltac2_simple_intropattern_clos:55,ltac2_typ:55,ltac2_type0:55,ltac2_type1:55,ltac2_type2:55,ltac2_typevar:55,ltac2val:[17,55],ltac:[5,13,24,25,35,38,43,52,53,57,58,59,60,62,63,64,66,67,71,74,77],ltac_expr0:[11,54],ltac_expr1:[54,66],ltac_expr2:[54,66],ltac_expr3:[3,29,54,58,64,66],ltac_expr4:54,ltac_expr:[5,9,11,29,54,55,60,62,64,66,71],ltac_production_item:71,ltacprof:17,ltb:[5,17,27,59],ltnv:57,luca:17,lui:77,lukasz:17,lumsdain:17,luna:24,luo:24,luttik:77,lv97:[3,77],lv:[17,51],lvar:7,lw11:[17,77],lxor:[17,59],lxor_comm:59,lyng:17,lyon:[24,77],lysxia:17,m0:[31,42,67],m150:58,m151:58,m1:[17,35],m2:[17,35],m:[0,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],ma:77,mac:[53,60],maccagnoni:17,machin:[10,17,24,25,27,32,36,51,54,55,64],machineri:[3,17,57],maco:[17,51,52],macro:[17,24,46,66,75],made:[2,3,14,17,24,29,34,35,38,41,46,51,53,54,55,57,58,64,66,71,72,75],magic:[2,17,24,55,59],mahboubi:[11,17,42,57,77],mai:[2,3,4,5,8,9,10,12,13,14,15,17,24,25,26,27,28,29,31,32,33,34,35,37,38,40,41,42,43,44,46,50,51,52,53,54,55,57,58,59,60,62,64,66,67,71,72,73,74,75,77],mail:17,maillard:17,main:[2,8,9,11,13,17,25,27,29,34,40,41,52,53,54,55,57,60,64,71],mainli:[14,60,75],maintain:[9,13,17,39,46,51,53,57,58,71],maintaint:17,mainten:[17,25,58,63],major:[15,17,24,26,42,51,53,55,73,74],makariu:17,makarov:[5,17],make:[2,3,4,5,8,9,10,11,12,13,14,17,24,25,26,27,28,29,30,32,33,34,35,37,38,39,41,42,43,44,45,46,51,52,53,55,57,58,59,60,62,64,66,67,71,75,77],make_a_le_b:14,make_b_lt_c:14,make_change_arg:17,makecmdgo:53,makefil:[17,51,52,53],malecha:17,malici:[17,51],maman:17,man:[25,51],manag:[3,13,17,24,25,32,38,51,53,57,59,60,62,73],mandatori:[2,8,17,32,57,66,71],mangin:17,mangl:[17,51,58,66],mani:[3,11,13,14,17,24,25,27,29,33,34,35,39,42,51,52,53,54,55,57,58,60,64,66,71,73],manifestli:35,manipul:[3,9,10,17,24,25,34,37,39,55,57,63,77],manna:24,manner:[10,24,51],manouri:24,mantissa:27,manual:[2,11,24,25,29,50,52,53,57,60,66,67,71],map2_ext:17,map:[2,3,5,13,17,24,25,26,27,34,35,36,39,41,44,51,53,57,58,59,60,71,72,75],map_append:17,map_const:17,map_eq_app:17,map_eq_con:17,map_ext:17,map_ext_foral:17,map_ext_in:17,map_id:17,map_last:17,map_length:17,map_map:17,map_morph:3,map_repeat:17,map_rev:17,map_shiftin:17,mapl:24,maplemod:24,mapsto:11,marc:17,march:[17,24,77],marech:17,marel:17,margin:[17,57],mari:17,mario:17,mark:[2,12,17,24,31,35,37,38,41,44,51,52,53,54,55,57,59,60,64,66,71],marker:[17,59],marshal:17,marti:17,martin:[17,24,27,34,77],martinez:17,mask:[2,35],massiv:35,master:[8,17,52,53,71,77],master_kei:57,match:[0,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,32,33,35,36,38,39,41,42,43,44,45,47,48,49,50,51,52,53,56,58,59,60,61,62,63,64,65,66,67,68,69,70,71,72,73,74,75,76,77],match_failur:[17,57],match_hyp:54,match_kei:54,match_pattern:54,matches_go:17,matej:17,materi:[17,24,25,50,57],math:[17,75,77],mathbb:[5,7,17],mathcal:[0,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],mathcomp:17,mathemat:[5,17,24,25,29,34,37,51,52,57,64,66,75,77],mathematica:24,mathematician:17,mathematiqu:77,mathieu:77,mathit:[5,26,34],mathrm:[0,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],mathsf:[0,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],mathtt:5,matsushita:17,matt:17,matter:[17,37,51,57,64,67],matth:17,matthew:17,matthia:17,matthieu:[3,9,14,17,77],matur:24,mauni:24,max:[14,17,24,39,46,54,59],max_comm:59,max_int:2,max_length:27,maxim:[3,13,17,25,41,51,57,71,77],maximum:[13,17,27,46,60,62,64,66],mayb:64,mayero:24,mbox:[0,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],mcb00:[67,77],mcbride:[67,77],md5:17,md:[17,71],mean:[2,3,5,9,10,11,12,13,14,17,24,25,26,27,28,29,31,32,34,35,38,40,42,43,44,46,51,52,53,54,57,58,59,64,65,66,71],meaning:[17,29,52],meaningless:75,meant:[2,3,14,17,55,59,64],meantim:17,meanwhil:17,measur:[9,17,34,54,72],measure_induct:17,mechan:[2,3,4,9,10,13,17,24,25,29,34,38,41,46,51,52,53,55,59,64,65,66,71,72,77],medium:57,meerten:6,meet:[2,9,71],melquiond:17,mem:[17,53],member:[13,42,55],memo:24,memoir:24,memori:[8,11,17,24,25,29,51,53],memprof:17,menial:57,mental:67,mention:[2,3,14,17,24,26,34,39,44,46,51,54,57,58,60,64,66,71],menu:[17,24,52,66],mere:[2,17,55,57,64,71],merg:[17,44],mergesort:17,merlin:[17,53],mess:17,messag:[3,4,8,11,12,13,14,16,17,24,26,28,29,30,34,35,37,40,41,42,43,44,46,51,52,54,55,57,58,59,60,62,64,66,67,71,74],met:53,meta:[17,24,25,39,53,59],metadata:[53,59],metalanguag:17,metamathemat:[24,77],metaprogram:54,metasyntact:55,metasyntax:17,metatheori:57,metavari:[17,24,25,54,55,62],method:[2,3,5,6,7,9,11,13,17,24,27,29,30,34,36,42,43,53,54,55,57,58,59,60,64,66,72,77],methodolog:[24,57],metric:17,metzger:17,meven:17,micaela:24,michael:17,michel:[17,24],micro:52,micromega:[17,25,61,66],micromega_core_plugin:[5,11,27,29,36,54,55,57,60,66],micromega_plugin:[5,11,27,29,36,54,55,57,60,66],microsoft:17,mid:17,middl:[17,29,54,57,71,75],might:[2,3,5,13,17,46,51,53,55,57,62,64,67,71,72,75],migrat:17,milad:17,mileston:17,miller:17,milner:[24,55,77],mimic:[13,37,57],mimram:17,min:[17,24,59],min_comm:59,mind:52,mingw:17,minic:24,minim:[8,17,24,25,34,51,53,57,67],minimum:17,miniorderedtyp:17,minki:17,minor:[17,51,57,71],minor_heap_s:51,minu:[11,17,27,29,41,72],minus_ind:72,minus_ipr:17,miquel:24,mirai:17,mirror:17,misc:[17,24,52],miscellan:25,mishandl:17,mislead:[17,71],misleadingli:17,mismatch:[17,46,53],misord:17,mispars:60,miss:[5,10,13,17,24,35,43,51,52,55,57,58,62,64,71,75],misspel:[46,59],mistaken:75,mistyp:10,misus:66,mitchel:77,mitig:[17,57,73],mix:[14,17,24,27,42,54,57,71],mixin:42,mixtur:24,mk_field:11,mk_linear:11,mk_rt:11,mk_sfield:11,mk_srt:11,mkmorph:11,mkpow_th:11,mkpredtyp:17,mkr:17,mkrat:37,mkrel:57,mkrmorph:11,ml4:17,ml:[3,5,6,8,9,11,17,24,25,26,27,29,34,36,42,43,46,51,52,53,54,57,58,59,60,63,64,66,72,77],mldep:17,mlg:[53,59],mli:[5,17,53],mlihtml:17,mllib:[17,53],mlpack:[17,53],mn:17,mod1:[35,51],mod2:[34,35],mod:[0,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],mod_abs_r_mod:17,mod_diveq_iff:17,mod_id_iff:17,mod_mod_abs_r:17,mod_mod_divid:17,mod_mod_opp_r:17,mod_opp_mod_opp:17,mod_opp_r_mod:17,mod_pow_l:17,mod_smal:17,mod_zmod:17,moda:[0,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],modal:17,mode:[9,13,14,17,24,25,29,30,32,34,38,41,46,51,54,58,59,60,65,75],model:[11,17,24,57,77],modern:54,modif:[2,4,11,17,36,41,58,71],modifi:[3,4,8,11,13,14,17,24,25,29,36,38,41,51,52,54,55,57,58,64,66,67,71],modimp:[0,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],modnam:57,modtyp:[0,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],modu:58,modul:[2,3,5,7,9,10,11,13,17,24,25,27,28,29,32,33,36,37,38,40,41,42,44,51,52,54,55,57,58,59,60,64,66,67,71,72,75],modular:[2,17,24],module_bind:35,module_expr_atom:35,module_expr_inl:35,module_prefix:53,module_typ:35,module_type_inl:35,modulenam:75,modulo:[2,4,5,11,17,24,27,34,54,57,58,59,71],modulu:17,moh86:[24,77],mohr:[24,27,77],mohrin:24,moin:17,moment:[17,26,52,53,54],mon_car:14,mon_op:14,mon_unit:14,monad:[14,17,55],monat:[17,24],monin:[17,24],monoid:[14,55],monoid_op:14,monoids_monoid:14,monolith:[2,17],monom:17,monomi:[5,11],monomorph:[9,17,25,27,29],mononorph:14,monospac:17,monoton:[3,4,17],monotoni:3,montevideo:24,month:17,moor:24,mora:77,moral:34,more:[2,3,4,5,6,8,9,10,11,12,13,14,17,24,25,26,27,28,29,30,31,33,34,35,36,38,40,42,44,46,51,52,53,54,55,57,58,59,60,62,63,64,66,67,71,72,73,74,75],moreov:[3,5,17,28,44,46,51,52,57,62,71],morgan:17,morph0:11,morph1:11,morph_add:11,morph_eq:11,morph_mul:11,morph_opp:11,morph_sub:11,morphism:[4,11,17,25,59,71],morphisms_prop:[3,17],morphisms_rel:17,morri:24,most:[2,3,4,10,12,17,24,27,29,34,38,41,45,46,51,52,53,54,55,57,58,60,63,64,66,67,71,72,73],mostli:[2,3,17,24,52,57,60],mot_to_ot:17,motiv:[11,17,55,57,77],motzkin:17,mous:[24,52],move:[13,17,24,25,43,52,53,55,66,67,71],move_loc:55,movement:[17,58],mset:17,msetavl:17,msetrbt:17,msg:55,msub:35,mt13:[42,77],mt:35,mtac2:63,mtac:55,mto:[0,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],much:[2,11,13,17,25,33,51,53,57,59,63,64,71],mul1g:57,mul:[2,5,17,27,36,52,57,59,71],mul_add_distr_l:6,mul_comm:[11,59],mul_exp:57,mul_reg_l:17,mul_reg_r:17,mul_spec:[27,36],mulder:17,mule:57,mulg1:57,mulgi:57,muln0:57,muln1:57,muln:57,mult1_rev:57,mult:[11,17,24,26,27,57],mult_comm:57,mult_ipr:17,mult_mark:57,mult_n_o:27,mult_n_sm:[27,59],multi1:57,multi1_rev:57,multi2:57,multi3:57,multi:[13,17,25,52,54,55,66,75],multi_goal_match0:17,multi_match0:17,multi_match:17,multibyt:17,multimatch:17,multipl:[2,3,4,9,14,17,24,25,27,29,34,35,40,44,52,58,59,60,64,66,67,71],multipli:[2,27,57],multirul:57,multiset_eq:3,multisuccess:17,mun94:[62,77],munch:17,murthi:24,museum:25,must:[2,3,4,6,7,9,10,11,12,13,14,17,24,25,26,27,29,30,34,35,36,37,39,40,41,44,51,52,53,54,55,57,58,59,60,62,64,66,67,71,72,74,75],mutabl:17,mutat:17,mutual:[9,17,24,25,29,30,32,37,54,55,67,71,72],my:[52,53,57,59],my_:40,my_congr_properti:57,my_def:57,my_eq:57,my_lemma1:57,my_lemma2:57,my_nat:40,my_o:40,my_package_plugin:59,my_scop:17,my_tac:52,my_tauto:54,my_tauto_ex1:54,my_tauto_ex2:54,my_toplevel:53,mybool:41,mybool_scop:41,myclass:37,mycod:53,myconst:24,myconstr:55,mye86:[66,77],myer:[66,77],myfield2:37,myfield:37,myfil:53,myfirst:54,myforal:71,mygeneratedfil:53,mylemma:57,mylet:71,mylib:74,myop:57,mypackag:53,myproj:53,myrecord:37,mytac:[17,55,57],mytauto:54,n0:[2,9,31,46,57,58,67,72],n1:[2,9,34,53,57,72],n2:54,n2bv_gen:17,n2bv_size:17,n2z:17,n:[0,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,68,69,70,71,72,73,74,75,76,77],nO:[0,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],n_1:[11,26],n_2:11,n_gt0:57,n_i:57,n_k:26,n_scope:71,n_sn:27,naddord:17,naiv:57,nake:57,name:[2,3,4,5,6,8,9,10,11,13,14,17,25,26,27,28,29,31,32,34,36,38,39,40,41,42,43,44,46,51,52,53,55,57,58,59,60,64,67,71,72,74,75],name_go:66,nameless:[17,77],nameofthem:52,namespac:[10,14,17,35,42,53,59],naming_intropattern:[58,67],nan:[17,27,71],nanci:24,nanevski:77,nant:17,narasimhan:[24,77],narboux:17,narith:[11,17,27],narithr:[11,17],narrow:[59,67],naryfunct:17,nash:17,nat2z:57,nat:[0,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,28,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],nat_cas:[27,67],nat_case_nodep:67,nat_compar:17,nat_compare_alt:17,nat_double_ind:27,nat_eq:42,nat_eqcl:42,nat_eqti:42,nat_ind:[27,34,58],nat_it:17,nat_l:42,nat_lecl:42,nat_leq_compat:42,nat_leqmx:42,nat_leqti:42,nat_leti:42,nat_of_int:2,nat_op:44,nat_or_id:57,nat_or_var:[5,13,17,54,58,60,67],nat_rec:[27,34,44,67],nat_rec_nodep:67,nat_rect:[2,27,34,59],nat_rect_plu:59,nat_scop:[6,27,31,34,38,46,57,71],nat_setoid:42,nat_sind:[27,34],nati:53,natint:17,nativ:[2,5,10,12,24,25,36,51,55,58,59,64],native_cast_no_check:58,native_comput:[17,25,32,36,51,58],native_compute_profil:64,nativecomput:[17,64],natnod:34,natord:17,natpair:17,natr:24,nattre:34,nattree_ind:34,nattree_rec:34,nattree_rect:34,nattree_sind:34,natur:[2,5,7,9,13,14,17,24,25,26,27,28,29,30,34,35,37,39,40,42,44,46,52,53,57,58,59,62,64,66,71,72],naveen:17,navig:[17,24,52,57,75],nawrocki:17,nbinari:[17,53],ncring:17,ncring_tac:17,nd:77,ndefop:17,ndigit:17,ndist:17,ndoubl:17,ne_:71,nearest:[17,27,54],nearli:73,necess:17,necessari:[3,4,9,13,17,24,29,31,33,37,53,55,57,59,62,64,67,71],necessarili:[4,46,67,72],necessit:24,need:[2,3,5,8,9,10,11,13,14,17,24,25,28,29,31,32,34,35,38,41,42,43,44,46,51,52,53,54,55,57,58,59,60,62,64,66,67,71,73,75,76],needless:60,neg:[5,17,27,29,30,37,64,66,71],neg_infin:27,neg_zero:27,negat:[17,27,54,57,58,60,62,67],negb:[5,13,27,62,71],negp:57,negpp:17,neither:[10,14,17,46,54,55,57,64,67],nelson:62,neq0:57,neq:11,neq_symmetr:59,neqb:13,neqb_implicit:13,nest:[3,9,17,24,25,29,32,35,38,40,54,57,58,59,64,66,71,75],net:17,network:60,never:[2,13,14,17,24,35,41,42,44,51,54,55,57,58,60,64],nevertheless:[2,17],new_goal:17,new_var:17,newcommand:[0,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],newdestruct:[17,24],newer:17,newest:[7,54,55],newinduct:[17,24],newli:[17,60,67],newlin:[17,24,29,53,54,71,75],newman:[17,24],newn:54,next:[3,9,13,17,24,27,29,33,34,42,44,46,51,52,54,55,57,60,64,65,66,67,71],next_down:27,next_up:27,ngan:17,nge0:57,ngt0:57,ni:53,nia:[17,25],nice:[52,57,67,75],nicer:17,nichola:17,nick:17,nickolai:17,nicola:[3,17,77],nicolo:17,niel:17,niesi:77,nijmegen:[17,24],nikishaev:17,nikita:17,nikolao:17,nil2:34,nil3:34,nil:[0,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],nil_spec:17,nilhl:[0,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],niln:46,nilw:34,ninf:27,niqui:17,niso:17,nix:17,nlist:71,nm:57,nmake:17,nmake_gen:17,nmax:17,nmin:17,nminu:17,nnn:[17,71],nnormal:27,nnumber:17,noccur_between:17,noccurn:17,nocor:[17,60],nocycl:53,node:[0,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],nodebug:17,nodup:17,nodup_app:17,nodup_app_remove_l:17,nodup_app_remove_r:17,nodup_concat:17,nodup_filt:17,nodup_iff_forallordpair:17,nodup_incl:17,nodup_incl_nodup:17,nodup_list_decid:17,nodup_map_nodup_forallpair:17,nodup_permutation_bi:17,nodup_rev:17,noedit:66,noi:[17,51],noinit:[17,29,51,66],noinlin:2,nois:53,nomacintegr:17,nomatch:[17,41],non:[2,4,6,8,9,10,13,14,17,24,25,26,27,28,29,30,35,37,40,41,46,51,52,53,57,59,60,62,64,66,72,75],nonassoci:71,nonconst:7,noncrit:17,noncumul:[17,25,29],none:[4,5,13,17,24,27,34,40,42,46,51,54,55,57,66,71],nonempti:60,nonetheless:[2,17,30,32,36,51,66],nonlinear:17,nonneg:60,nonprimit:17,nonproptyp:17,nonrecurs:[17,37,40,67,72],nonreflex:25,nonsimple_intropattern:55,nonstandard:17,nonsymmetr:25,nontermin:[17,29,54,55,71],nontrivi:[11,17,46,51,57],nonuniform:[4,17],nonzero:[3,11,37,54],nor:[10,11,17,26,34,35,46,51,52,53,54,55,57,58,59,64,67,71],norec:51,norm:11,normal:[2,3,4,5,11,17,24,26,27,29,30,31,34,35,41,44,51,52,53,54,55,57,59,64,66,67,71,72,77],normfr_mantissa:27,norp:57,north:77,nosimpl:57,not_1_ipr:17,not_eq_:27,not_eq_sym:27,not_found:[17,24],not_i:34,not_i_i:34,not_ipr:17,not_locked_false_eq_tru:17,not_nodup:17,nota:17,notabl:[10,17,24,37,51,55,57,64,67],notat:[4,5,9,10,11,14,24,25,26,28,29,31,33,34,35,36,37,38,40,41,45,46,51,52,53,57,58,60,64,67,73,74,75,77],notation_declar:71,notconst:11,notcresolut:[17,57],note:[2,3,4,5,7,8,10,11,12,13,14,15,17,24,26,27,28,29,34,35,37,40,41,42,43,46,51,52,53,54,55,57,58,59,60,62,64,66,67,71,72,74,77],notempl:17,notepad:53,noth:[3,17,38,41,51,54,55,57,58,62,64,66,67],notic:[3,4,5,17,26,34,35,38,46,51,52,54,57,58,64,66,71,72,74],notin:[17,26],notin_flat_map_foral:17,notin_remov:17,notion:[5,11,17,24,25,26,27,33,34,46,51,54,55,58,64,71,77],nott:[17,27],notypeclass:[17,58],nouniv:54,nov:24,novel:[17,25],novelti:[17,25],novemb:[17,24,77],novic:[17,57],now:[2,3,4,11,13,14,17,24,26,27,30,34,35,41,42,46,51,52,53,54,55,57,59,60,64,67,71,72,74],np_n:34,npe:11,npeano:17,npo:37,nq:67,nra:[17,25],ns:[0,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],nsatz:[17,25,61],nsatz_comput:17,nsatztact:[7,17],nset:71,nsi:17,nsubn:27,nsucc_doubl:17,ntf:51,nth:[17,27,58],nth_append_l:17,nth_append_r:17,nth_error:17,nth_error_:17,nth_error_app:17,nth_error_con:17,nth_error_cons_0:17,nth_error_cons_succ:17,nth_error_ext:17,nth_error_firstn:17,nth_error_map:17,nth_error_nil:17,nth_error_o:17,nth_error_repeat:17,nth_error_rev:17,nth_error_seq:17,nth_error_skipn:17,nth_ext:17,nth_middl:17,nth_nth_nth_map:17,nth_order:17,nth_order_ext:17,nth_order_hd:17,nth_order_replace_eq:17,nth_order_replace_neq:17,nth_order_tl:17,nth_repeat:17,nth_replace_eq:17,nth_replace_neq:17,ntn:24,nullstellensatz:[5,7,17],num1:24,num2:24,num:[11,17],numarg:24,number:[2,3,4,5,7,8,11,13,14,17,24,25,26,29,30,34,36,37,39,40,41,42,43,44,46,52,53,55,57,58,59,62,64,66,67,72,74,77],number_modifi:71,number_or_str:[29,71],number_string_via:71,numer:[5,11,17,24,27,29,59,71],numgoal:[17,25],nuprl:24,nvar:24,nw:2,ny:77,nz:17,nzdomain:17,nzero:27,nzmulord:17,nzmulorderprop:17,nzprop:17,nzproperti:17,o:[0,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],o_:[27,37],oapp_comp:17,obei:[17,24,37],obfusc:59,obindeapp:17,obj:[2,24,42],object:[2,3,4,8,9,11,13,14,17,24,25,26,28,29,30,31,33,35,37,38,39,40,41,42,44,51,53,55,57,59,64,67,71,72],oblig:[13,17,25,37,57,62,72],observ:[17,34,37,40,54,55,59,66,71],obsolet:[6,17,24,51,58],obstacl:[17,42],obstruct:57,obtain:[2,3,4,5,17,34,36,54,55,57,58,64,67,72,75],obviou:[3,34,57,71],obvious:17,ocaml:[2,11,17,24,25,27,29,32,36,51,53,54,55,63,64,66,71,73,75],ocaml_librari:53,ocamlbuild:17,ocamlc:17,ocamldep:17,ocamldoc:75,ocamlfind:[17,53,59],ocamllib:53,ocamlopt:17,ocamlrunparam:[17,51,66],ocamlwarn:53,ocan_comp:17,ocan_in_comp:17,occ:57,occ_switch:57,occas:17,occasion:[17,24,29,53,66],occs_num:[17,55,58,64],occur:[2,3,4,8,17,24,26,28,30,34,37,38,41,42,44,46,54,55,57,58,59,60,64,66,67,71],occur_between:17,occurn:17,occurr:[2,3,11,14,17,24,25,26,43,44,46,52,54,55,59,60,64,71],octal:17,octob:[24,77],ocurr:58,odd:[0,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,68,69,70,71,72,73,74,75,76,77],odd_:34,odd_alt:17,odd_alt_odd:17,odd_even:[17,67],odd_even_ind:17,odd_ind:[34,67],odd_j:57,odd_odd:17,odd_sind:[34,67],odditi:54,oddn:57,oddt:17,oddt_event_rect:17,of_bit:59,of_constr:55,of_float:36,of_goal:17,of_hex_uint:59,of_int63:27,of_int64:36,of_int:[17,36],of_intro_pattern:17,of_list_to_list_opp:17,of_module_typ:35,of_nat:[17,57],of_num_uint:[29,59,71],of_preterm:17,of_str:55,of_typ:[4,17,28],of_type_inst:[17,34,37],of_uint:[59,71],of_uint_dec:71,off:[2,8,10,12,13,14,17,24,27,29,34,35,37,43,44,46,51,52,53,54,57,59,64,66,67,71],offer:[17,29,46,51,52,54,57,59,71],offici:[17,54],offset:[17,27,53],offsid:17,ofil:53,often:[2,3,10,13,14,17,25,28,43,46,52,53,54,55,57,58,66],ok:[17,29,52,58],okada:17,okj:17,old:[3,11,24,25,51,53,55,58,60,66,67],older:[17,29,51,67],oldest:[4,17],oldf:55,oldroot:17,olift:17,olift_comp:17,oliv:17,olivi:[17,24],omap_comp:17,omapeapp:17,omapebind:17,omega2:17,omega:[17,24],omegalemma:17,omegatact:17,ominu:11,omiss:17,omit:[2,3,8,14,17,27,28,29,30,32,34,37,38,40,41,42,44,45,46,53,54,55,57,58,59,60,66,67,71,75],omnisci:17,onc:[3,8,9,10,11,13,14,17,24,25,27,32,34,41,42,44,46,51,53,55,57,58,59,60,64,66,67,71,72],ondemand:[17,51],one:[2,3,4,5,6,8,9,11,12,13,14,15,17,24,26,27,28,29,30,31,33,34,35,36,37,38,40,42,43,44,46,51,52,53,54,55,57,58,59,60,62,63,64,66,67,71,72,74,75,77],one_goal_match0:17,one_minus_one_is_zero:36,one_pattern:[13,59,60],one_term:[3,5,7,11,13,29,34,54,58,60,62,64,67,71,72],one_term_with_bind:[3,58,64,67,72],one_two_ir:37,one_typ:[29,58,64],ones:[2,3,4,6,8,13,14,17,25,28,34,35,37,44,46,52,53,54,57,58,59,63,66,67,71,75],ones_0:17,ones_succ:17,ongo:[17,63],onli:[2,3,4,5,6,7,8,9,10,11,12,13,14,17,24,25,26,27,28,29,30,31,32,33,34,35,37,38,39,40,41,42,43,44,46,50,51,52,53,54,55,57,58,59,60,62,64,66,67,71,72,73,74,75],onlin:[27,73],onto:[17,71],oop:17,op1:[57,58],op2:58,op:[5,42,44,53,57,66,71],opac:[17,59,64],opam:[17,25,27,73],opam_packag:53,opaqu:[3,6,8,9,14,17,24,25,31,32,35,38,51,57,59,60,64,66,67,71,75],opcod:17,open:[3,5,6,11,13,17,25,27,35,36,38,42,50,52,54,55,57,59,60,64,66],open_bind:[6,28,58,64],open_constr:[17,55,71],open_constr_flag:17,open_constr_with_bind:17,openbsd:17,opencont:[25,50],openpub:[25,50],oper:[3,5,9,10,11,14,17,24,25,27,32,34,36,51,52,54,55,57,60,64,66,67,71],operand:[17,27,64],operation:36,operators_properti:17,opl:5,oplt:5,oplu:11,opn:58,opp:[17,27],oppen:62,opportun:17,oppos:[17,57],opposit:[17,31,32,46,58,64],opt:[17,24,53,55,71],optim:[5,9,17,24,25,36,58,64,66,77],optimis:24,optimize_heap:[17,66],option:[5,8,9,10,11,13,14,16,24,25,26,27,34,35,38,40,42,44,46,50,52,53,54,55,57,58,59,60,62,64,67,71,74],option_eqb:13,option_eqb_obligation_1:13,option_eqb_obligation_2:13,option_eqb_obligation_3:13,option_ind:[27,34,58],option_rec:[27,34,58],option_rect:[27,34,58],option_sind:[27,34,58],oq:77,or_and_intropattern:58,or_assoc:59,or_ind:[34,40],or_introl:[27,34,40,46,58,67],or_intror:[27,34,40,46,58,67],or_sind:[34,40],oracl:5,orang:52,orb:[2,27,57,62],orb_comm:59,orb_negb_l:17,ord:[13,57],ord_ind:57,ord_rec:57,ord_rect:57,ord_sind:57,order:[2,3,4,6,7,8,9,11,12,13,14,15,17,24,25,26,27,29,30,32,34,35,37,40,42,43,46,51,52,53,54,55,57,60,61,62,64,66,67,71,72,75,77],ordered_set_lang:53,ordered_typ:[17,60],orderedgrammar:71,orderedtyp:[17,60],orderedtypeex:17,orderg1:57,orderg:57,orderg_dvd:57,ordersex:17,orderstac:17,ordinari:[3,17,26,37,39,71],org:[25,50,64,75,77],organ:[17,24,25,53,54,57],organis:24,orient:[17,24,25,51,54,55,57,60,64],oriented_rewrit:[55,64],origin:[2,3,4,9,11,17,24,29,31,34,38,43,44,46,53,57,58,62,64,66,67,71],orp:57,orphan:53,orphan_foo_bar:53,orpp:17,orsai:[17,24],orthogon:57,os:[17,53],oscar:17,ot:60,other:[2,3,4,5,8,9,10,11,12,13,14,24,25,26,27,28,29,30,31,32,33,34,35,36,37,38,41,42,43,51,52,53,54,55,57,58,59,60,62,63,64,67,71,72,76],other_const:42,otherwis:[2,3,9,13,14,17,28,29,34,41,42,44,46,51,52,53,54,55,57,58,59,62,64,66,67,71,73],otim:11,our:[4,5,7,11,17,24,34,35,54],ouri:77,ourselv:[14,34],out:[8,17,24,29,42,52,53,54,57,58,59,60,66,71,75],outcom:[17,51,53,54,67],outdat:17,outer:[14,17,46,66],outermost:67,outperform:17,output:[2,3,4,11,14,17,24,33,42,51,52,53,54,59,60,64,66,71,75],output_valu:17,outputst:17,outsid:[3,5,9,11,12,13,14,17,28,29,35,38,40,41,42,43,53,54,59,60,66,71],ouvert:77,over:[2,3,11,14,17,24,25,26,27,28,30,32,34,37,38,39,40,41,42,44,46,52,53,54,58,59,60,61,62,64,66,67],overal:[51,54,64,75],overflow:[2,17,59,66,71],overhaul:17,overhead:[17,53,64],overlap:[5,17,42,46,53,57,59,66],overli:17,overlin:[0,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],overload:[17,24,25,71],overrid:[2,14,17,37,51,53,57,66,67,71],overridden:[17,27,54,57,71,75],overriden:17,overview:[17,25,71],overwrit:[52,64,66],overwritten:75,ovl:[0,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],ow:55,own:[5,10,17,24,25,35,42,44,54,57,59,60,62,66,67,75],owr:77,p0:[9,31,67,72],p1:[13,17,37,57,67],p2:[37,57,67],p2q:57,p:[0,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],p_0:5,p_1:[5,7,34,35],p_2:[5,35],p_:[7,34],p_i:[7,34],p_j:[5,34],p_l:34,p_m:34,p_p:34,p_r:[34,35],p_rmin:17,p_u:34,p_unit:54,p_xy:57,pa:57,pab:57,pablo:17,pack:[3,42,53],packag:[17,24,25,35,42,51,52,59,67,73,75],packtyp:14,pad:57,page:[17,25,27,51,52,71,75],pain:57,pair:[0,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],pair_eq:42,pair_eqcl:42,pair_eqti:42,pair_l:42,pair_lecl:42,pair_leq_compat:42,pair_leqmx:42,pair_leqti:42,pair_leti:42,pairusualdecidabletypeful:17,pairwis:57,palaiseau:17,palat:[17,55],pale:66,palmskog:17,pane:52,panel:[8,17,52,66],panic:55,paolo:17,paper:[13,24,42,54,57,72,77],par95:[9,77],par:[8,17,52,54],paradigm:24,paradox:[34,77],paragraph:[11,27,35,40,57,75],paral:17,parallel:[17,24,25,38,51,52,53,54,57,76],param:17,param_1:17,param_n:17,paramet:[3,4,5,7,8,13,14,17,24,25,28,29,34,37,40,41,43,44,53,54,55,58,59,60,64,66,67,71,72],parameter:[3,5,11,14,17,24,25,28,37,40,54],parametr:[17,24,25,34,40,64],parent:[9,17,24,77],parenthes:[2,3,8,17,24,28,29,35,37,46,54,55,57,58,67,71],parenthesi:[17,57,66],pari:[17,77],parimala:17,parith:[17,27],pariti:17,parm:71,parrai:[17,36],pars:[9,17,25,27,29,41,42,46,51,54,57,59,60,74,75],parse_entri:17,parser:[14,17,24,29,53,71],parsimoni:57,part:[2,3,10,11,13,15,17,24,25,27,29,34,35,37,46,51,52,53,54,55,57,58,66,67,71,72,73,74],parti:[17,51,52,53,59,75],partial:[3,13,17,24,34,35,37,44,51,53,54,57,59,62,66,71,72],particip:[17,57],particular:[2,3,6,9,10,12,13,17,29,30,31,32,33,34,37,38,40,42,52,53,54,55,57,59,60,64,66,71,75],particularli:[17,25,42,51,53,64,71],partit:17,partition_as_filt:17,partli:[17,57],partner:17,pascal:17,pass:[3,5,8,10,12,17,24,37,38,42,51,52,53,54,55,57,60,64,66,67,71,75],past:[2,17,52,64],pat1:17,pat:[17,55],patch:17,patenaud:17,path:[2,4,5,17,24,25,27,35,51,52,54,60],pathnam:[51,53],patholog:2,patn:17,patrick:[11,24],pattern0:[28,40],pattern10:40,pattern1:40,pattern:[2,9,13,17,24,25,27,28,30,32,34,40,41,42,45,60,64,67,72,77],pattern_occ:[58,64],paul:17,paulin:[17,24,27,34,77],paulson:24,pautomata:24,pave:17,payload:27,pb:57,pc:11,pcan_in_comp:17,pcan_in_inj:17,pcm:17,pcompar:17,pcoq:24,pdf:[17,29,77],pe:11,peadd:[5,11],peak:[17,53,66],peano:[17,24,25,34,57,60,71],peano_dec:24,peanonat:[6,17,58,59],pec:[5,11],pedant:59,peeval:11,pemul:[5,11],pen:57,pennsylvania:[17,77],peopl:17,peopp:11,pepow:11,per:[2,3,11,17,24,52,53,57,59,71],per_symmetr:59,percentag:54,perf:[17,64],perfectli:2,perfetto:51,perform:[2,3,5,7,8,11,13,17,24,25,26,34,41,42,46,51,54,55,57,60,62,64,66,67,71,72],perfum:17,perhap:[52,53,58],period:[17,24,29,52,54,60,66,74],perm:54,perm_append:54,perm_aux:54,perm_con:54,perm_ind:54,perm_refl:54,perm_sind:54,perm_tran:54,permiss:[17,53],permit:[9,17,24,25,34,37,38,53,54,55,58,60,64,66,67,71],permtat:17,permut:[3,17,25,55,57],permutation_app:17,permutation_app_inv_m:17,permutation_app_middl:17,permutation_app_rot:17,permutation_app_swap_app:17,permutation_con:17,permutation_count_occ:17,permutation_elt:17,permutation_elt_map_inv:17,permutation_exist:17,permutation_flat_map:17,permutation_foral:17,permutation_forall2:17,permutation_imag:17,permutation_incl_cons_inv_r:17,permutation_ind_transp:17,permutation_list_max:17,permutation_list_sum:17,permutation_map_inv:17,permutation_map_same_l:17,permutation_middle2:17,permutation_morph_transp:17,permutation_permutation_transp:17,permutation_pigeonhol:17,permutation_pigeonhole_rel:17,permutation_refl:17,permutation_repeat:17,permutation_transp:17,permutation_transp_con:17,permutation_transp_equiv:17,permutation_transp_sym:17,permutation_vs_cons_cons_inv:17,permutation_vs_cons_inv:17,permutation_vs_elt_inv:17,permutsetoid:17,perri:17,persist:[9,17,24,29,35,36,38,64,77],person:[24,64],perspect:[24,77],pertain:54,pervas:17,pesub:11,peter:[17,24],peterson:17,pex:[5,11],pexpr:11,peyton:77,pf_type_of:17,pf_unsafe_type_of:17,pfen:[17,24,77],pff:8,pfst:14,pg:[17,66],pgdn:17,pgivesbound:8,pgup:17,phantom:42,phantom_ind:42,phantom_rec:42,phantom_rect:42,phantom_sind:42,phase:[17,24,52,54,55,57,64,72],phd:[24,77],phi:17,philosoph:11,phoni:[17,53],phrase:[25,71],physic:[17,24,35,51,53,59,75],physical_dir:24,phyumn5ooqtymh4h6i0nsskchnaysu:51,pi:[13,17,52],pi_:28,pichardi:[72,77],pick:[17,42,51,52,53,57,58,66,67],pictur:17,pide:17,pident:14,piec:[11,42,43,53,55,57],piecewis:17,pierc:17,pierr:[2,17,24,77],pile:57,pinf:27,pinj:11,pink:52,pinot:17,pinpoint:57,pioneer:24,pipe:17,pise:24,pit:17,pittsburgh:77,pivot:5,pk:[14,57],pkg:[53,59,75],pl:55,place:[2,3,17,32,40,43,51,53,57,58,59,64,66,67,71,75],placehold:[17,43,44,51,57,58,66,71],plai:[2,17,26,42,64,66],plain:[9,17,35,57,75],plainli:55,plan:[10,17,25,53,55,72],plane:[17,24,25],platform:[17,24,36,51,53,54,72],pleas:[17,24,44,53,54,55,62,66,67,72,77],plu:[0,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],plug:59,plugin:[2,5,11,12,17,24,25,29,33,35,53,54,55,59,63,66,71,72],plugin_tutori:[17,63,74],plumb:67,plural:[17,28,38],plus0l:60,plus0r:60,plus1:71,plus_assoc_reverse_stt:59,plus_equ:[57,72],plus_fct:41,plus_ind:[57,72],plus_ipr:17,plus_n_o:[27,59],plus_n_sm:[27,59],plus_o_n:59,plus_rec:[57,72],plus_rect:[57,72],plus_sn_m:59,plussl:60,plussr:60,pm89:[24,77],pm93a:[31,77],pm93b:[24,77],pm:57,pmult:17,pmult_comm:17,pn:[13,17,57],pnormal:27,po:[17,24,59,71],point:[2,3,11,13,17,24,25,26,27,32,34,35,36,39,51,52,53,54,55,57,66,71],pointer:[24,26],pointless:57,pointwis:3,pointwise_rel:3,pol:11,polici:[17,57,74],pollack:24,polylist:24,polymorph:[2,3,13,17,24,25,26,27,29,30,31,32,33,37,39,40,41,44,46,51,59,66,67,71],polynom:11,polynomi:[5,7,17,24,25,61],ponen:58,pool:[17,62],poor:17,poorli:[43,54],pop:[57,71],popl:77,popul:29,port:[3,17,24,55,72],portegi:17,portion:[17,57],pos_neg_int63:71,pos_sub:17,pose:[5,17,24,34,54,55,57,58,67],posit:[3,4,5,7,9,10,11,14,17,24,25,27,30,36,37,39,41,44,46,51,52,54,55,57,58,59,64,66,67,71],position:[2,58],positive_as_ot:17,positive_scop:[27,71],positiveint:55,positivstellensatz:[17,25],posreal:17,possibl:[2,3,4,5,8,9,11,13,14,17,24,27,28,31,34,35,37,41,42,43,44,46,51,52,53,54,55,57,58,59,60,64,66,67,71,73,74,75],post:[17,24,53,57],postfix:[17,57,71],postpon:[17,58,66],postprocess:11,postscript:75,postul:28,potenti:[9,13,25,42,46,52,54,55,57,67,71],pottier:[7,17,24,57],poulin:17,poulsen:17,pow:[5,17,27,59],pow_div_l:59,pow_inv:17,pow_ipr:17,pow_lower_bound:17,pow_n:11,pow_po:[17,71],power:[4,5,11,17,24,27,54,57,67,71,72],power_theori:11,powerrz:17,powerrz_inv:17,powerrz_mult:17,powerrz_neg:17,powerset:34,pp:[17,53],ppair:14,pphi_dev:11,pphi_dev_ok:11,pplu:10,pplus_rewrit:10,ppm89:[24,77],pprod:14,pqequiv:57,pr1:14,pr2:14,pr:17,pr_numgoal:54,pr_p:57,practic:[2,3,5,17,24,25,32,34,39,42,53,55,57,58,64,66,71,74,77],pre:[2,17,25,53,60],preambl:75,preced:[17,25,27,29,46,54,57,58,60,66,75],preceed:64,precis:[4,8,13,17,24,26,29,31,33,34,35,37,39,46,51,57,64,71],precisionnotzero:8,precompil:[17,25,51,64],precondit:58,pred:[9,17,27,54,57,59,60,64],pred_add:64,pred_class:17,pred_doubl:17,pred_n:17,pred_oapp:17,pred_sn:27,pred_sort:17,predecessor:27,predefin:[11,24,25,51,52,66],predic:[3,9,17,24,25,26,27,30,34,40,42,54,60,64,77],predict:[14,17,54,64],predtyp:17,preexist:17,prefac:60,prefer:[7,17,25,34,51,53,57,58,59,62,66,71],preferenti:71,prefix:[2,3,9,11,14,17,24,27,28,34,35,38,40,41,42,44,51,52,54,57,58,59,64,66,67,71,75],preformat:75,preimag:17,preliminari:11,prelud:[2,17,25,29,51,59,66],premis:[17,24,28,35,57,60,66],prenex:57,preomega:17,preorder:[13,57,59],preorder_reflex:[13,59],preorder_transit:13,prepar:[17,24],prepend:[51,53,66],preproccess:17,preprocess:[11,17],preprocessor:[11,24],prerequisit:[17,53],presburg:24,prescrib:[17,57],presenc:[8,17,24,34,44,46,57,64,72],present:[2,3,6,9,11,13,15,17,24,25,26,29,30,32,33,34,37,41,42,44,45,46,50,53,54,55,57,58,59,60,61,63,64,65,66,67,71,73,74,75,76],preserv:[2,5,14,17,24,25,29,30,34,42,55,57,64,67,71],press:[52,77],pressur:60,presum:[17,71],presuppos:[5,75],preterm:[9,17,55],pretti:[17,24,25,27,51,53,57,59,71],pretyp:[17,51,55],prevail:34,prevent:[13,17,29,34,41,42,51,53,54,57,64,71],preview:[2,52],previou:[2,3,4,8,9,11,13,15,17,24,27,29,31,34,37,40,41,42,45,46,51,52,54,55,57,59,60,62,64,66,67,71,74],previous:[2,13,17,28,34,38,52,54,57,59,71],prf_equiv:42,prim2sf:[27,36],prim:[17,71],primari:[52,54],primarili:[32,34,58,66],prime:[3,17,29,34,57],prime_decomp:57,prime_i:57,primfloat:[17,27,36,59,71],primfloatnot:17,primint63:[36,59,71],primit:[2,10,12,13,14,17,24,25,30,33,34,41,46,54,55,57,64,67],primstr:[27,36,71],primstringaxiom:27,princ:17,princeton:17,princip:[17,24,34,57,72,77],principia:24,principl:[2,5,17,24,25,27,30,34,37,51,57,58,63,64,71,77],print:[2,5,6,8,11,12,13,17,24,25,27,29,31,34,35,36,38,39,41,42,51,52,53,57,58,60,62,64,66,67,74],print_list:55,printabl:71,printconf:59,printer:[17,24,29,46,57,59,71],printf:17,prior:[17,51,54],prioriti:[13,17,37,46,52,57,59,66,71],prisqu:17,privat:[13,14,17,25,29,30,34,37],private_:[17,59],probabl:[2,17,32,44,51,54,57,58,59,75],problem:[2,4,7,9,13,17,24,29,34,42,44,46,51,52,53,54,58,62,66,67],problemat:[40,55],proc:77,proce:[3,11,13,52,57,71],procedur:[3,4,11,17,24,25,54,57,60,62,64,77],proceed:[58,77],process:[9,11,14,17,24,25,26,30,32,35,41,42,51,52,53,55,57,58,59,60,64,66,67,75,76],processor:[17,27,36],prod:[2,17,26,27,34,46,62,67],prod_:57,prod_appvect:17,prod_curri:17,prod_curry_uncurri:17,prod_eqb:13,prod_eqb_obligation_1:13,prod_f_r0:17,prod_f_so:17,prod_ind:[27,34],prod_length:17,prod_monoid:14,prod_of_sigt:17,prod_rec:[27,34],prod_rect:[27,34],prod_sigt_prod:17,prod_sind:[27,34],prod_uncurri:17,prod_uncurry_curri:17,prodimp:26,prodt_curri:17,prodt_uncurri:17,produc:[2,5,7,8,9,11,13,14,17,24,25,29,32,34,36,38,40,41,44,52,53,54,55,57,64,66,71,72,73,74,75],product:[2,3,5,10,11,13,14,17,24,26,27,28,34,36,39,40,46,54,55,57,59,60,64,66,67,71],prof:[17,53],profil:[5,17,25,53,59,64],program:[0,1,3,4,5,7,8,10,11,12,13,14,15,16,17,18,19,20,21,22,23,24,25,26,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,56,57,58,59,61,62,63,64,65,66,67,68,69,70,71,72,73,74,75,76,77],program_branch_0:[9,13],program_branch_1:[9,13],program_branch_2:13,program_scop:17,program_simpl:9,programm:[3,24,25,65],programmat:13,progress:[3,17,24,25,51,52,55,60,66,77],progress_evar:17,proj1:[27,66],proj1_sig:[17,46,57],proj2:27,proj:[17,24,54],project:[2,3,9,10,12,13,14,15,17,24,25,27,29,30,34,40,41,42,51,52,54,55,57,59,60,64,72,73,74,76],projections2:27,projs1:24,projs2:24,projt1:[17,27],projt2:27,projt3_eq:17,prolog:[17,24,60],prompt:[17,24,52,54,59],prone:[54,57],proof:[2,3,6,7,9,11,13,17,24,26,27,29,30,33,34,36,37,38,39,40,42,43,44,51,52,53,55,59,61,62,64,67,72,73,74,75,76,77],proof_admit:17,proof_irrelev:34,proofgener:53,prooftre:[17,59,66],proofview:55,prop:[0,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,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],propag:[3,11,17,41],propbinop:5,proper:[3,9,17,24,54,55,59,67],proper_prf:17,properli:[2,8,9,10,17,29,52,53,57,59,66],properti:[3,4,6,9,11,12,13,17,24,25,26,27,30,31,32,34,38,39,42,45,46,57,58,67,72,77],propextension:17,propop:5,proport:64,propos:[17,24,34,54],proposit:[2,3,5,10,17,24,25,26,28,29,30,31,32,33,34,39,40,51,57,58,62,64,66,67,77],propositionnel:77,propr:24,propuop:5,prose:17,protect:[11,17,30,57],protocol:[17,77],protonmail:17,prototyp:[9,17,24],provabl:[5,11,17,34,39,57,58,66],prove:[3,5,7,8,9,11,17,24,25,27,30,32,34,35,42,43,57,58,60,62,64,72,77],proven:[11,17,52,58,64,66,67],prover:[4,5,15,17,24,26,29,31,33,52,55,59,65,73,75,76],provid:[2,5,6,7,8,9,10,11,12,13,14,15,16,17,24,25,26,27,29,30,32,33,34,35,36,37,41,42,43,44,51,52,53,54,55,57,58,59,60,62,63,64,65,66,67,71,72,73,74,75],provis:62,prune:[38,57],ps:75,psatz:[17,25],psatzadd:5,psatzc:5,psatzin:5,psatzmul:5,pseudo:[17,57,60],psnd:14,pstring:[27,36],psubn:27,publi:77,public_nam:53,publicli:17,publish:[24,53,77],puech:17,puf:77,pull:[17,55],pun:[17,55],punctuat:[71,75],pure:[3,7,11,17,55,57,64,71,72,75],purifi:17,purpos:[12,14,17,24,27,34,35,42,51,52,54,55,57,59,64,66,67,71],push:[2,17,57,71],put:[3,5,13,14,17,34,35,43,51,53,54,57,58,59,60,66,67,71,72,75],putnam:24,puydt:17,puzzlement:24,pv:[9,77],pwd:[2,14,59],px:[11,24,57],py:17,python2:17,python3:17,python:[17,53],pzero:27,q1:[5,10,13,46,57],q2:[5,10,57],q2p:57,q2r:[5,57],q3:57,q4:57,q:[2,3,5,7,10,11,12,17,24,27,34,35,46,51,53,54,55,57,58,59,67,71,75],q_1:[7,34],q_:7,q_factordenom:17,q_factornum:17,q_factornum_l:17,q_i:[7,34],q_l:34,q_occurr:55,q_orient:55,q_r:34,q_reduce_fl:17,q_rewrit:55,q_scope:[5,71],q_u:34,q_with_bind:55,qarchimedean_power2_po:17,qarchimedeanexp2_po:17,qarith:[5,17],qarith_bas:17,qc:71,qc_scope:71,qcanon:11,qden:17,qden_cancel:17,qed:[3,5,6,8,9,12,13,14,17,24,29,32,34,36,38,40,42,51,52,54,57,58,59,60,62,64,66,67,72],qeq_from_part:17,qeval_formula:5,qextra:17,qhyp:55,qinv_neg:17,qinv_po:17,qinv_swap_neg:17,qinv_swap_po:17,qle_neq:17,qlt_leneq:17,qm:13,qmicromega:5,qmult_frac_l:17,qmult_inject_z_l:17,qmult_inject_z_r:17,qmult_le_lt_compat_po:17,qmult_lt_le_compat_nonneg:17,qnum:17,qnum_cancel:17,qopp_lt_compat:17,qpower_0_lt:17,qpower_1_l:17,qpower_1_le_po:17,qpower_1_lt:17,qpower_1_lt_po:17,qpower_decomp:17,qpower_decomp_po:17,qpower_le_1_increas:17,qpower_le_compat:17,qpower_le_compat_inv:17,qpower_le_compat_l:17,qpower_le_compat_l_inv:17,qpower_lt_1_increas:17,qpower_lt_compat:17,qpower_lt_compat_inv:17,qpower_lt_compat_l:17,qpower_lt_compat_l_inv:17,qpower_pos_lt:17,qr:46,qreduce_l:17,qreduce_num_l:17,qreduce_r:17,qreduce_zero:17,qround:17,qtautocheck:5,qtautochecker_sound:5,quad:5,quadrat:[2,17],qualid:[2,4,5,10,11,13,14,17,29,35,37,39,40,41,42,46,51,54,55,57,59,60,62,64,66,67,71,72,74],qualid_annot:[28,29,44],qualifi:[2,17,24,25,28,32,38,51,53,54,55,57,58,59,64,66,71],qualiti:[10,14,17],quantif:[2,3,4,13,14,17,24,26,27,28,60,67],quantifi:[8,14,17,24,25,26,28,34,39,44,57,58,62,67],quarkcool:17,quasi:57,quentin:17,queri:[13,17,25],query_command:[29,59,64],query_extra_dep:59,question:[25,34,54,55,57,60,66],quick:[13,17,24,27,54,57,66,74],quickli:[16,17,25,44],quicksort:24,quiet:75,quinn:17,quirk:52,quit:[2,3,11,13,17,25,34,42,54,55,57,60],quo_rem_un:57,quodlibet:[17,58],quot2:17,quot:[2,5,13,17,24,25,28,29,44,51,55,59,66,71,75],quot_rem:17,quot_rem_to_equ:[5,17],quotat:[17,24,25,66,75],quoted_str:53,quotient:[2,5,17,40,57,64],qux_plugin:53,qwit:5,qzero_eq:17,r0:[5,17],r1:[3,5,17,27,41,44,57,59],r2:[3,17,27,41,44,57,59],r3:57,r4:57,r:[2,3,5,7,9,11,13,14,17,24,27,28,34,35,37,41,44,51,53,54,57,58,59,60,64,67,71,72,75,77],r_1:3,r_2:3,r_dist:17,r_forest_size_complet:72,r_forest_size_correct:72,r_ifp:17,r_inj:17,r_item:57,r_pattern:57,r_plus_complet:[57,72],r_plus_correct:[57,72],r_prefix:57,r_s_inv:28,r_scope:[11,27,71],r_sqr:24,r_step:57,r_tree_size_complet:72,r_tree_size_correct:72,ra:13,rab:27,rabs_inv:17,race:17,raci:17,radboud:17,radd:11,radd_0_l:11,radd_assoc:11,radd_sym:11,radicalmax:7,radix3:71,radix3_ind:71,radix3_rec:71,radix3_rect:71,radix3_scop:71,radix3_sind:71,radix:[8,66],radixmorethanon:8,radixmorethanzero:8,radixnotzero:66,radziuk:17,railroad:24,railroadcross:24,rais:[2,3,10,13,17,29,35,54,55,64,72],raise_nat:10,rakam:[17,64],ralf:17,ralph:17,ram:17,ramachandra:17,ramkumar:17,ran:54,ranalysi:[17,24],ranalysis_reg:17,rand:17,randi:24,random:17,randomli:17,rang:[5,17,26,29,52,55,58,71],range_selector:54,rappli:[17,58],rard:77,rare:[11,17,66],rasmusson:17,rat:37,rat_bottom_nonzero:37,rat_irreduc:37,ratan:17,rather:[5,11,13,17,24,29,30,34,35,53,54,55,57,58,59,64,67,71],ratio:24,ration:[7,17,24,25,37,61,71],rational:[17,55,57],rauglaudr:[17,24],raw:[2,14,17,54,55,71],raxiom:17,rb:13,rbase:[11,17,24],rbox:12,rc:[17,24],rceil:5,rcl:34,rcomput:24,rdefinit:17,rdist:17,rdistr_l:11,rdiv:[3,5,27],rdiv_0_l:17,rdiv_0_r:17,rdiv_1_l:17,rdiv_1_r:17,rdiv_def:17,rdiv_diag:17,rdiv_diag_eq:17,rdiv_diag_uniq:17,rdiv_eq_compat_l:17,rdiv_eq_compat_r:17,rdiv_eq_reg_l:17,rdiv_eq_reg_r:17,rdiv_mult_distr:17,rdiv_mult_l_l:17,rdiv_mult_l_r:17,rdiv_mult_r_l:17,rdiv_mult_r_r:17,rdiv_neg_neg:17,rdiv_neg_po:17,rdiv_opp_l:17,rdiv_opp_r:17,rdiv_pos_cas:17,rdiv_pos_neg:17,rdiv_pos_po:17,re:[17,24,29,32,38,46,51,52,53,54,55,58,59,60,64,66],reach:[13,52,58],reachabl:71,reactiv:[8,17,59],read:[15,17,26,29,42,51,52,57,59,64,71,75],readabl:[2,17,24,29,53,57,64,71,75],reader:[3,11,24,29,31,42,57],readi:[17,51,57,60],readili:53,readm:[24,71],real:[2,3,7,11,24,25,34,46,53,55,66,67,71],realfield:11,realist:[2,42],realiz:[24,25,27,32],realli:[17,32,57],reappli:9,reason:[2,3,5,9,10,11,17,24,25,34,44,51,53,54,55,57,59,62,65,71,72,75,77],rebind:[5,17,52],rebuild:[13,17],rebuilt:53,rec:[2,17,24,35,54,55,75],recal:[46,55,64],recaptur:17,recdef:72,recent:[3,24,25,53,71],recheck:66,recip:[17,53],recogn:[2,4,5,8,11,17,24,29,34,46,51,52,55,62,67,71,75],recognit:[17,75],recommend:[4,8,13,14,15,17,32,35,46,51,52,53,54,55,57,58,59,60,64,66,67,72,74,75],recompil:[17,51,52,53,59,64],recomput:[34,53],reconstruct:[37,46],record:[2,3,8,10,11,12,13,14,17,24,25,30,33,34,42,54,55,57,59,60,62,67,71],record_definit:[4,13,30,34,37],record_field:[37,42],recov:[3,8,14,17,30,46,51,54,67],recover:55,recoveri:[8,17,52],rect:67,rectyp:17,recurr:25,recurs:[2,5,9,17,24,25,31,32,33,37,40,41,44,46,51,53,54,57,58,59,60,64,66,67,75,77],recursor:[2,17],red:[8,17,51,52,54,64,66],red_expr:[3,17,32,54,64],red_flag:17,redeclar:[13,17],redefin:[4,17,54,55,57,66,71,75],redefinit:[17,54,55],redesign:[17,24],redex:[2,17,25,31,34,64,71],redflag:17,redirect:[17,51,59,75],redo:[17,57,67],reduc:[3,7,8,10,11,12,13,17,24,26,31,32,34,36,37,40,41,44,51,53,57,58,59,60,64,66,67,71],reduce_and_try_to_solv:54,reduct:[2,3,9,10,11,12,17,25,26,30,32,36,41,44,46,51,53,57,58,67,77],redund:[17,24,43,46,57],redux:2,ref:[17,59],refactor:[17,64],refer:[2,3,4,5,8,10,13,14,16,24,25,28,29,31,32,34,35,36,37,38,39,41,42,44,46,50,51,52,53,55,57,58,60,62,64,66,67,71,72,74,75],referenc:[2,17,53,71],reference_occ:64,refglob:55,refin:[6,13,14,17,24,27,30,32,34,35,38,43,46,52,54,55,57,58,66,71],refl:[3,17],refl_eq:24,refl_equ:[3,17,57],reflect:[9,11,14,17,24,25,27,40,52,53,62,64,66,72,77],reflect_fals:57,reflect_tru:57,reflectf:40,reflectt:[40,57],reflex:[3,5,6,11,13,17,24,27,34,36,51,54,57,59,60,62,64,66,67,71],reflexion:24,reflexive_eq_dom_reflex:59,reflt:46,refman:17,refold:[17,64],reform:17,reformat:17,refrain:17,refresh:71,refrom:[17,51],refus:[2,3,64],refut:[25,57],regard:[3,14,17,51,58],regardless:[14,17,42,57,60,66],regener:53,regexp:[17,60],region:57,regist:[2,3,4,5,7,9,11,13,17,25,32,42,57,64,67,71,72],registr:[2,17,25],regress:17,regroup:17,regular:[9,10,13,17,36,46,51,55,57,60,64,75],regularli:17,rehaul:24,reifi:[5,17],reific:[7,17,64],reimplement:17,reimport:71,reinfer:44,reintroduc:[17,57],reject:[9,17,26,34,57,64,67,71],rel:[2,14,17,26,27,35,51,53,55,59,71],relat:[5,6,7,9,10,11,13,14,17,24,25,26,27,31,34,35,40,41,42,44,51,52,53,57,58,59,60,64,67,71,72,75],relation_definit:[3,13,17,59],relation_oper:17,relationclass:[3,17,64],relationship:[17,29],relaunch:17,relax:[2,17,30,44,53,57,60],releas:[13,15,17,24,25,52,53,57,63,74],releg:24,relev:[12,17,24,28,30,32,34,40,46,51,53,54,57,58,64,66,71],reli:[5,17,24,30,32,33,34,38,46,51,52,53,54,55,57,58,59,64,66,67,71],reliabl:17,relianc:17,reliev:24,reload:[51,52,59],reloc:24,relpr:17,rem:[5,17],remain:[2,3,9,11,13,14,17,24,34,36,39,41,42,44,46,52,57,58,64,66],remaind:[17,34,55],remap:71,remark:[4,17,24,25,32,34],remedi:[5,17],rememb:[17,52,57,58,75],remi:17,remind:[2,3,57],remot:17,remov:[2,3,4,5,11,14,17,24,29,31,37,41,46,51,52,53,55,57,58,59,60,66,67,71,72,74,75],remove_app:17,remove_con:17,remove_concat:17,remove_incl:17,remove_length_l:17,remove_length_lt:17,remove_remove_comm:17,remove_remove_eq:17,removelast_firstn_len:17,removelast_last:17,remzi:17,renam:[2,17,24,25,34,37,55,57,58,59,71,74],renard:[3,24],render:[17,24,75],renewcommand:75,renn:77,reopen:52,reorder:[17,25,52],reorgan:17,repair:[12,17],repars:[17,54],repeat:[3,17,25,43,44,52,55,57,58,59,66,67],repeat_app:17,repeat_con:17,repeat_eq_app:17,repeat_eq_con:17,repeat_eq_elt:17,repeat_to_concat:17,repeatedli:[17,31,57,71],repect:58,repetit:[25,54,60],replac:[2,3,4,7,9,10,11,17,24,25,28,31,32,34,37,41,43,44,46,51,52,53,54,55,57,58,59,62,64,66,67,71,74,75],replace_append_l:17,replace_append_r:17,replace_id:17,replace_replace_eq:17,replace_replace_neq:17,replace_with:55,replai:[11,57],replic:57,repo:53,report:[4,8,12,17,24,29,52,54,55,59,64,72,77],repositori:[17,53,63,74],repr:17,repres:[2,3,5,11,13,14,17,24,26,27,28,29,31,32,34,36,37,39,40,42,43,51,52,53,54,55,57,58,59,64,65,66,67,71],represent:[2,3,5,11,12,17,24,27,29,34,37,51,53,57,64,71],reprint:[17,66],reprocess:[52,54],reproduc:44,req:11,req_dec_t:17,req_em_t:17,request:[3,14,17,25,43,51,64],requir:[2,3,5,6,7,8,9,10,11,13,14,17,24,27,28,29,30,31,32,34,35,36,38,42,43,44,51,52,53,54,55,57,58,59,60,62,63,64,66,67,71,72,73,74,75],required_vo:51,rerun:5,resack0:60,research:[24,77],resembl:57,reserv:[17,25,27,29,35,40,54,57,59],reserv_list:44,reset:[2,17,24,29,30,34,40,41,46,51,52,54,59,72],resg0:60,resg1:60,residu:[17,57],resili:[17,25],resilient_command:17,resiz:17,resolut:[3,13,17,24,25,58,60,66,71,75],resolv:[9,13,14,17,35,43,52,55,57,58,59,60,64,66,67,71],resolve_tc:17,resort:[43,52,54,55,67],resourc:51,resp:[5,17,34,36,46,57],respect:[2,3,4,5,11,13,14,17,24,26,27,30,34,38,40,42,44,52,54,55,57,58,59,60,64,66,67,71,72,74,75],respons:[2,10,17,52,55,75],rest:[2,3,13,17,26,27,29,36,42,52,57,66],restart:[17,51,52,53,54,57,66],restart_tim:[17,54],restor:[17,29,54,57,66],restrict:[2,3,12,14,17,24,26,34,35,40,51,54,57,58,59,60,62,67,71],restructur:[17,24],result:[2,3,4,5,8,10,11,12,13,14,17,24,26,27,31,32,34,39,40,42,44,46,51,52,53,54,55,57,58,59,60,62,64,66,67,71,75],resum:17,ret:54,retain:17,retract:17,retri:54,retriev:[17,51,54,59,60,77],retro:17,retyp:17,reunion:77,reus:[14,17,41,57,58,59,63,64,66],reusabl:25,rev:[27,71],rev_con:17,rev_eq_app:17,rev_inj:17,rev_length:17,rev_nil:17,rev_repeat:17,rev_rev:17,rev_shiftin:17,revamp:17,revers:[7,15,17,25,27,34,41,57,58,60,66],reverse_coercion:[4,17],reversecoercionsourc:4,reversecoerciontarget:4,revert:[17,52,57,58,59],revgoal:17,review:[2,17,27],revis:[17,24,55],revisit:67,revolutionari:24,rew:[17,67,77],rew_iff_rev:57,rework:17,rewrit:[6,11,14,17,24,25,33,34,35,52,54,55,58,59,60,61,77],rewrite_occ:[3,64],rewrite_rul:10,rewrite_strat:[3,17],rewriterel:[3,17,57],rewritten:[3,9,11,24,30,46,57,58,64],rewrot:[11,17],rewstrategi:[3,17],rewstrategy0:3,rewstrategy1:[3,17],rexists_between:17,reynald:17,rfloor:5,rfrom:[17,51],rfunction:24,rgb:51,rge:[17,27],rge_gt_or_eq:17,rge_gt_or_eq_dec:17,rge_l:17,rge_lt_dec:17,rge_refl:17,rgeom:24,rgt:[17,27],rgt_le_dec:17,rgt_minus_po:17,rgt_or_l:17,rgt_or_not_gt:17,rh:[17,55,57,59],ri:[11,17,51],ribbon:52,rich:[9,17,57,73],richard:17,richer:[13,25],ricki:17,rid:[9,17,54,57],rideau:[17,57],rieg:17,rifrom:[17,51],right:[0,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,47,48,49,50,51,52,53,54,55,56,57,58,59,60,61,62,63,64,65,66,68,69,70,71,72,73,74,75,76,77],righta:71,rightarrow:[5,7,26,75],rightarrow_:[11,37],rigid:[3,10,13,14,17,24,60,72],rigor:[2,24],rin:17,rineq:17,ring31:17,ring:[7,17,24,25,27,37,61,62],ring_eq_ext:11,ring_mod:11,ring_morph:11,ring_plugin:[2,3,5,9,11,27,29,36,42,43,54,55,57,58,59,60,64,66,72],ring_polynom:11,ring_simplifi:[11,17],ring_theori:11,ringer:17,ringmicromega:5,rinv:[5,27],rinv_0_lt_contravar:17,rinv_div:17,rinv_eq_compat:17,rinv_eq_reg:17,rinv_inv:17,rinv_lt_0_contravar:17,rinv_mult:17,rinv_mult_simpl:17,rinv_neg:17,rinv_opp:17,rinv_po:17,rinv_r_simpl_l:17,rinv_r_simpl_m:17,rinv_r_simpl_r:17,ripault:17,rise:[13,24],risk:[10,17,24,51,59,66],rl:34,rle:[17,27],rle_epsilon:17,rle_gt_dec:17,rle_half_plu:17,rle_lt_or_eq:17,rle_or_gt:17,rle_or_not_l:17,rle_rinv:17,rlength:17,rlist:17,rlogic:17,rlt:[17,27],rlt_0_2:17,rlt_0_minu:17,rlt_ge_dec:17,rlt_half_plu:17,rlt_minus_0:17,rlt_monotony_contra:17,rlt_monotony_rev:17,rlt_or_g:17,rlt_or_not_lt:17,rlt_rminu:17,rmin_cas:17,rminu:[5,27],rminus_def:17,rminus_diag:17,rminus_eq_0:17,rminus_eq_compat_l:17,rminus_eq_compat_r:17,rminus_gt_0_lt:17,rminus_plus_distr:17,rminus_plus_l_l:17,rminus_plus_l_r:17,rminus_plus_r_l:17,rminus_plus_r_r:17,rmp:58,rmul:11,rmul_1_l:11,rmul_assoc:11,rmul_sym:11,rmult:[5,11,27],rmult_div_assoc:17,rmult_div_l:17,rmult_div_r:17,rmult_div_swap:17,rmult_gt_reg_r:17,rmult_inv_l:17,rmult_inv_m_id_r:17,rmult_inv_r:17,rmult_inv_r_id_l:17,rmult_inv_r_id_m:17,rmult_inv_r_uniq:17,rmult_neg_cas:17,rmult_neg_neg:17,rmult_neg_po:17,rmult_pos_cas:17,rmult_pos_neg:17,rmult_pos_po:17,rnm:58,ro:11,road:17,roadmap:17,robbert:17,robbiano:77,robert:[17,77],robin:[17,77],robinson:24,robust:[2,17,51,57,60,66,75],robustli:64,rocq:[3,4,6,8,9,10,11,12,13,14,15,17,24,26,28,29,30,31,32,33,34,35,36,37,38,41,42,43,44,45,46,50,52,54,55,58,59,62,63,64,65,66,67,73,76],rocqlib:59,rocquencourt:[17,24],rodi:17,rodolph:17,roi:[54,62,77],role:[17,26,33,42,55,71,75],romain:17,romega:[17,24],root:[3,17,25,27,46,51,59],ropp:[11,27],ropp_def:11,ropp_div:17,ropp_div_distr_l:17,ropp_eq_reg:17,ropp_minus_distr:17,ropp_neg:17,ropp_po:17,roquencourt:24,ros98:[9,77],rosetta:54,rosser:77,rotat:[24,54,57],round:[5,17,27,53],rousselin:17,routin:2,roux:17,row:[17,46],rplu:[5,27],rplus_0_l_uniq:17,rplus_eq_0:17,rplus_eq_r0:17,rplus_ge_reg_r:17,rplus_gt_reg_r:17,rplus_int_part_frac_part:17,rplus_le_lt_0_neq_0:17,rplus_minus_assoc:17,rplus_minus_l:17,rplus_minus_r:17,rplus_minus_swap:17,rplus_neg_lt:17,rplus_neg_neg:17,rplus_neg_npo:17,rplus_nneg_g:17,rplus_nneg_nneg:17,rplus_nneg_po:17,rplus_npos_l:17,rplus_npos_neg:17,rplus_npos_npo:17,rplus_pos_gt:17,rplus_pos_nneg:17,rplus_pos_po:17,rplus_sqr_eq_0_l:17,rpow:11,rpow_pow_n:11,rpower:17,rr:77,rrika:17,rs:17,rs_r:17,rsa:24,rsigma:24,rsqr:17,rsqr_def:17,rsqr_div:17,rsqr_inv:17,rstar:[17,24],rstep:57,rstrength:17,rsub:11,rsub_def:11,rta:77,rtac:55,rtauto:[17,62],rtran:58,rtrigo:24,rtrigo_calc:17,rudi:17,rudimentari:71,rug:55,rule:[3,4,5,11,12,13,14,17,24,25,29,32,33,35,36,37,39,41,42,44,46,51,53,54,55,58,59,60,62,66,67,77],run:[2,5,8,9,13,14,17,24,25,29,51,53,57,59,60,64,66,71,73],runbox:12,runner:17,runtim:[17,51,55,73],rushbi:77,russel:[9,17,24],rusu:72,rw_head_pattern:10,rw_pattern:10,rw_pattern_arg:10,rwf:27,ryan:17,s0:[43,46],s1:[3,30,38,57],s2:[3,30],s754_finit:27,s754_infin:27,s754_nan:27,s754_zero:27,s:[0,1,3,4,5,6,7,8,9,10,11,12,13,14,15,16,17,18,19,20,21,22,23,24,25,26,28,29,30,31,32,33,34,35,36,37,38,39,40,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,68,69,70,71,72,73,74,75,76,77],s_1:[7,34,35],s_2:[34,35],s_3:35,s_:[7,34],s_i:[5,7,34],s_item:57,s_j:34,s_k:34,s_nat:4,s_o_plus_inr_depr:17,sacerdoti:[3,17,24],safe:[2,11,17,34],safeimplicit:2,safer:[17,24],safeti:2,sai:[2,3,4,17,24,26,27,28,29,31,34,42,52,53,54,55,57,58,64,71,74],said:[3,4,17,26,34,36,42,44,55,59,71],saikawa:17,sakaguchi:17,sake:[35,55,66,71],salient:[17,24],sam:[17,77],same:[2,3,4,6,8,9,10,11,12,13,14,17,24,25,26,28,29,30,31,34,35,36,37,38,40,41,42,43,44,51,52,54,55,57,58,59,60,62,64,66,67,71,72,75],samel:71,samuel:[11,17,24],san:75,sandrin:77,santiago:17,satifi:34,satisfi:[3,4,5,11,13,14,17,30,34,35,54,55,59,64,67,71],satur:[5,17],save:[8,11,17,25,35,51,53,57,66],saw:24,sc:24,scale:[17,24,51,57,64,71],scan:54,scene:57,schedul:17,schema:24,schemat:[52,57],scheme:[2,11,17,24,25,26,27,34,37,40,46,51,57,59,62,77],scheme_kind:67,scheme_typ:17,scherer:17,schneider:17,schommer:17,schroeder:24,scienc:[24,77],scientif:[24,77],scinart:17,scope:[5,11,17,24,25,27,29,32,36,38,42,43,45,52,54,55,57,59,60,64,66],scope_kei:[40,55,59,64,71],scope_nam:71,scott:[17,24],scratch:52,screen:[17,52,59],screenshot:[52,66],script:[5,8,17,24,25,35,42,43,53,54,55,57,58,59,60,63,64,66,73],scrupul:17,scrutine:17,sdf:77,seamlessli:53,search:[2,3,4,5,7,13,17,24,25,42,44,51,52,53,61,62,64],search_item:59,search_queri:59,searchabout:[17,24],searchhead:17,searchiso:24,searchpattern:[17,24],searchrewrit:[17,24],seassau:17,sebastiaan:77,sec:[53,54,64],second:[2,3,4,8,9,10,11,13,15,17,24,25,26,28,35,37,38,40,42,44,51,52,53,55,57,59,60,64,66,67,71,75],secondari:[52,53],secondli:[2,17],section:[3,5,6,7,8,9,10,11,12,17,24,25,26,27,28,29,30,31,32,33,34,35,36,37,40,41,42,43,46,51,52,53,54,55,57,58,59,60,64,65,67,71,74],section_path:59,section_var_expr0:66,section_var_expr50:66,section_var_expr:[60,66],secur:51,sed:17,see:[2,3,4,5,7,8,9,11,12,13,14,17,24,26,27,28,29,30,31,32,33,34,35,36,37,38,39,40,41,42,43,44,46,51,52,53,54,55,57,58,59,60,62,64,66,67,71,72,74,75],seem:[2,5,17,71],seemingli:71,seen:[2,4,13,14,17,24,32,34,55,57,67,71],seg:24,segfault:[10,17],segment:[2,17,24,52,59,71],seldin:77,select:[8,13,17,25,35,37,41,42,52,53,54,55,58,59,60,64,66,67,71,75,77],selector:[8,17,25,43,53,58,59,64,66],self:[14,17,54,55,67,71],selfid:14,selfpid:14,semant:[3,11,13,14,17,24,25,26,29,35,36,39,41,44,53,54,57,58,71,77],semeria:17,semi:[4,11,17],semi_field_theori:11,semi_morph:11,semi_ring_theori:11,semicolon:[52,53,57],semidecis:24,semifield:11,semir:[11,17],sempti:12,sempty_ind:12,sempty_rec:12,sempty_rect:12,sempty_sind:12,send:17,sens:[4,24,26,30,54,55,57,71],sensibl:[14,24],sensit:[17,24,29,59],sent:52,sentenc:[17,24,29,36,52,54,55,57,59,75],sentence_1:24,sentence_n:24,sep:71,separ:[2,3,10,14,17,24,25,26,29,33,34,35,40,44,46,51,52,53,54,55,57,58,59,67,71,74],septemb:[17,24,77],seq:[12,13,30,46,55,57,67],seq_:17,seq_ind:[12,46],seq_length:17,seq_rec:[12,46],seq_rect:[12,46],seq_sind:[12,46],seqseri:24,sequenc:[2,3,5,17,24,25,27,28,29,30,46,51,57,58,59,60,64,66,71,75],sequent:[54,57,58,62,77],sequenti:[17,54,55,58,64],sergei:17,seri:[25,27,29,35,54,57],serial:[58,67],serif:75,seriou:[17,71],serv:[17,24,25,26,40,55,57,60],server:[17,52],session:[2,14,17,51,52,59],set1:26,set2:26,set:[0,1,3,4,5,6,7,8,9,10,11,12,14,15,16,17,18,19,20,21,22,23,24,25,27,28,30,31,32,33,34,35,36,38,39,40,42,43,44,45,46,47,48,49,50,51,52,53,54,55,56,59,61,62,63,64,65,67,68,69,70,71,72,73,74,75,76,77],set_diff_nodup:17,set_eq:3,set_map:17,set_p:34,seth:17,setistyp:17,setoid:[7,10,11,17,24,25,42,57],setoid_:[3,17],setoid_reflex:17,setoid_replac:[17,24,64,71],setoid_rewrit:[3,17,24,60,64],setoid_symmetri:17,setoid_theori:[11,17],setoid_transit:17,setoidchoic:17,setoidlist:17,setoidpermut:17,setoidtact:[17,71],setting_nam:[29,51],setup:[17,25],seventh:77,sever:[2,3,4,5,11,17,24,25,26,28,29,30,31,32,34,40,42,44,46,51,52,54,55,57,59,60,64,65,67,71,72,75,76],sf64mul:[27,36],sf:72,sf_1_neq_0:11,sf_sr:11,sfclassifi:17,sfdiv_def:11,sfinv_l:11,sfst:12,shachar:17,shachnev:17,shade:52,shadow:[14,17,44,66],shaji:17,shall:[2,17,24,26,31,34,39,42,57,71],shankar:77,shao:77,shape:[2,3,57],share:[2,11,13,14,17,24,28,29,34,46,51,52,53,57,59,60,64,67,71],she:[24,55],sheet:75,shelf:[17,66],shell:[51,53,57,59,75],shelv:[6,13,17,25,43,57,58,60],shelve_unifi:[17,58],shen:17,shengyi:17,shenlebantongi:17,shift:[17,52,57],shiftl:17,shiftl_lower_bound:17,shiftr:17,shiftr_upper_bound:17,shine:57,shinnar:17,ship:[17,66],shiwei:17,shortcut:[13,17,25,52,55,64,71],shorten:[17,28],shorter:[17,31,35,57,59],shortest:35,shorthand:[17,41,54,57,64],should:[2,3,9,10,11,12,13,14,17,24,26,28,29,30,32,34,35,40,41,42,44,46,51,52,53,54,55,57,58,59,60,62,64,66,67,71,74],shouldn:[53,54,75],show:[2,3,5,7,8,9,11,13,14,17,24,25,27,34,35,37,38,42,51,52,53,54,57,58,59,60,64,67,71],show_profil:17,show_zifi:5,shown:[5,9,13,14,17,27,29,31,34,37,38,42,43,51,52,53,54,57,58,59,60,66,71,75],shrink:[17,66],shuffl:57,sibut:17,siddharth:17,side:[3,10,13,14,17,24,25,27,32,34,35,38,43,52,54,55,57,58,60,62,64,67,71],sig2:[17,27,35,67],sig2_ind:27,sig2_rec:27,sig2_rect:27,sig2_sind:27,sig:[2,17,27,28,35,67,71],sig_ind:27,sig_rec:27,sig_rect:27,sig_sind:27,sigact:77,sigint:17,sigma:[14,17,37,67,71],sign:[5,8,11,17,29,36,46,52,53,60],signal:[2,8,17,57],signatur:[2,3,11,17,24,34,35,54,55,59],signature_scop:17,signaturet:17,signific:[17,24,51,63,66],significantli:[11,17,24,57,66],sigplan:77,sigt2:[17,27,67],sigt2_ind:27,sigt2_rec:27,sigt2_rect:27,sigt2_sind:27,sigt:[17,27,67,71],sigt_ind:27,sigt_of_prod:17,sigt_of_sigt2:17,sigt_prod_sigt:17,sigt_rec:27,sigt_rect:27,sigt_sind:27,sigtnot:17,sigurd:17,sile:17,silenc:[4,17,24,41,46,57,62,74],silent:[12,14,17,24,29,51,53,59,66,72],similar:[2,3,5,9,13,17,24,26,27,34,35,37,38,51,53,54,55,57,58,59,60,62,64,66,67,72,74,75],similarli:[9,10,13,14,17,26,28,36,38,42,44,46,52,53,54,55,57,62,64,71,75],simon:[17,77],simonbouli:17,simpl:[3,4,10,11,17,24,25,29,37,41,42,43,46,52,53,54,57,58,59,60,62,67,72],simpl_depind:67,simpl_rel:[3,17],simple_bind:67,simple_intropattern:[17,55,58,67,71,72],simple_intropattern_clos:58,simple_occurr:[58,60,64],simple_reserv:44,simple_tact:[24,54],simpler:[17,24,57,58,62,64],simplest:[55,57],simplex:17,simpli:[3,4,11,13,14,17,24,31,39,54,55,57,59,62,67,71,75],simplic:[35,54],simplif:[2,11,17,24,25,41,54,67],simplifi:[2,11,17,24,41,54,57,64,67],simplify_dep_elim:67,simplify_eq:[17,24,67],simplify_typ:54,simplify_type_eq:54,simplist:42,simpson:24,simul:[3,17,24,57,66],simultan:[3,17,24,25,26,30,32,34,42,53,57,58],sin3pi4:17,sin:17,sinc:[2,3,4,5,8,10,11,12,13,14,17,24,26,28,30,34,35,37,41,42,44,46,51,52,53,54,57,58,59,60,66,67,71,74,75],sine:17,singhal:17,singl:[2,3,4,13,14,17,24,25,28,29,30,34,35,37,40,44,46,52,53,55,57,58,59,60,64,66,67,71,75],single_z_r_r1_depr:17,singleton:[2,13,17,24,34,54,58],sint63:[17,36],sint63_scop:36,siromonei:[24,77],site:55,situat:[3,4,11,17,46,54,57,71],sixth:17,sizabl:57,size:[2,3,9,13,17,24,34,37,51,52,55,57,59,64,71,72],sizef:34,sizet:34,skeleton:9,skip:[8,17,41,42,46,51,53,54,57,58,64,66,67],skipn:17,skipn_length:17,skipn_non:17,skipn_seq:17,skipn_skipn:17,slant:75,slash:[17,57],slave:51,slexprod:17,slider:52,slight:[2,17,24,58],slightli:[3,17,24,35,51,52,54,55,57,58,67],slow:[3,11,17,53,54,55],slowdown:17,slower:[17,51,60,62],slowest:53,slowli:54,slrnsc:17,small:[3,5,8,11,14,17,25,26,27,33,34,39,42,44,52,53,57,64],smaller:[3,11,14,17,32,33,34,53,58,62,67,72],smallest:[3,5,27,34,67],smart:17,smart_glob:71,smarter:17,smit:17,sml:24,smooth:[17,24,57],smorph0:11,smorph1:11,smorph_add:11,smorph_eq:11,smorph_mul:11,snd:[17,24,27,35,42,46,71],snd_list_prod:17,snippet:[55,75],snoc:67,snyke7:17,so08:[13,77],so:[2,3,4,7,8,9,10,11,12,13,14,17,24,26,27,29,31,32,34,35,36,37,38,44,46,51,52,53,54,55,57,58,59,60,62,64,66,67,71,73,74,75],societi:77,socket:17,soegtrop:17,soft:[25,72],softwar:[17,24,25,59,77],sogetrop:17,solut:[3,5,13,17,42,44,58,59,63,67],solv:[2,3,5,7,11,13,17,24,25,39,42,44,57,60,61,62,64,67],solvabl:[17,58,62],solve_constraint:66,solve_iso:54,solve_iso_ex1:54,solve_iso_ex2:54,solve_perm:54,solve_type_eq:54,solver:[9,17,25,65],some:[3,4,5,6,8,9,10,11,12,13,14,17,24,25,26,28,29,30,31,32,34,37,38,40,41,42,44,45,46,51,52,53,54,55,57,58,59,60,61,62,63,64,66,67,71,72,73,75],some_class:17,some_const:42,some_expr:17,some_term:17,somehow:46,someon:17,someth:[17,31,52,53,54,55,59,64],sometim:[14,17,24,25,31,34,46,53,54,55,57,59,60,66,67,71],somewhat:[55,64,71],soon:[8,9,17,24,42,52,54,57],sop:24,sophia:[17,24],sort:[0,1,2,3,4,5,6,7,8,9,10,11,12,13,15,16,17,18,19,20,21,22,23,24,25,26,27,28,29,30,31,32,33,35,36,37,38,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],sort_famili:[67,72],sortclass:[4,17,57,71],sorted_sort:17,sotaro:17,soubiran:17,sought:46,soukouki:17,sound:[2,17,34],sourc:[2,4,5,14,24,25,51,52,53,55,57,59,71,73],source_date_epoch:17,soz07:[9,77],sozeau:[3,9,14,17,77],sp1:17,space:[3,17,29,52,53,57,59,66,71,74,75],space_overhead:51,span:17,spanjel:17,spawn:[17,54],speak:[5,11],spec:[5,17],spec_float:27,special:[2,3,4,9,12,13,16,17,24,25,27,28,29,34,51,52,53,54,55,59,60,64,66,67,71,75],specialist:17,specif:[2,3,5,9,11,24,28,31,32,34,35,36,39,40,42,51,52,53,55,57,58,59,60,61,64,66,67,71,77],specifi:[2,3,4,5,6,9,11,13,17,24,25,27,28,29,32,34,35,36,37,40,41,43,44,46,51,52,53,54,55,57,58,59,60,62,64,66,67,71,72,75],spectacular:24,speed:[3,13,17,24,34,64],spell:17,spent:[17,51,53,54],sphinx:17,sphinx_rtd_them:17,sphinxcontrib:17,spin:17,spirit:[17,34,55],spite:17,spitter:17,spiwack:17,splay_ar:17,split:[2,17,25,27,29,34,42,51,54,57,58,60,66,67,75],split_combin:17,split_length_l:17,split_length_r:17,split_rab:27,split_rmult:27,splitabsolu:24,splitat:17,splitrmult:24,spontan:57,spot:55,spr1:12,spr2:12,spread:53,spring:24,springer:77,sprod:12,sprop:[0,1,2,3,4,5,6,7,8,9,10,11,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],spuriou:[4,17,57,71],spurious:17,sqrt:[17,27,59],sqrt_inv:17,sqrt_iter:59,squad:2,squar:[5,17,24,44,54,59,71,75],squash:[12,14,17],squash_ind:14,squash_prop_rect:14,squash_prop_srect:14,squash_sind:14,sr:10,sradd_0_l:11,sradd_assoc:11,sradd_sym:11,src:[4,53],srdistr_l:11,srefl:[12,46],sring_eq_ext:11,srinivasan:17,srmul_0_l:11,srmul_1_l:11,srmul_assoc:11,srmul_sym:11,ssig:12,ssnd:12,ssort:4,ssr:[17,57,59,66],ssr_binder:57,ssrautoprop:57,ssrbool:[17,57],ssreflect:[0,1,2,3,4,5,6,7,8,9,10,11,12,13,14,15,16,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,58,59,60,61,62,63,64,65,66,67,68,69,70,71,72,73,74,75,76,77],ssreflect_plugin:57,ssrewrit:17,ssrfun:[17,57],ssrhave:[17,57],ssrident:57,ssripat:57,ssripat_scop:57,ssrmatch:[17,57],ssrmatching_plugin:57,ssrnat:57,ssroldrewritegoalsord:57,ssrrewrit:57,ssrsearch:17,ssrsyntax:57,sstuff:4,stabil:17,stabl:[8,17,24,53],stack:[17,25,41,54,55,57,59,71],stage:[17,34,42,55,66],stai:[2,27],stale:17,stalmarck:[2,24],stand:[5,10,17,24,26,28,34,53,71],standalon:[17,51],standard:[2,3,5,9,14,25,29,35,36,40,51,52,53,54,58,59,62,64,65,66,67,72,73,74,75],stanza:53,star:[17,60,62],starred_ident_ref:66,start:[2,3,8,9,13,17,24,25,26,27,29,32,34,35,37,40,41,42,44,46,52,53,54,55,58,59,60,64,66,67,71,74,75],start_coq:53,start_profil:17,startclass:17,startup:[12,51,53,60],stat:66,state:[2,3,5,7,8,11,13,17,24,25,27,29,31,32,37,51,52,54,55,57,58,59,62,64,67,71],statement:[8,9,17,24,28,32,33,41,42,44,51,57,58,59,64,66,67,71],station:17,statist:[5,17,66],statu:[8,12,13,14,17,51,52,53,54,57,71],std:[17,55],stdlib:[2,3,5,6,9,12,14,17,27,28,35,36,51,53,54,55,57,58,59,64,66,67,71,75],stdout:[17,75],steckler:17,stefan:17,stell:17,stem:17,stengl:17,step:[3,5,7,11,13,17,24,25,26,29,41,51,52,53,54,58,60,64,65,67],stepanenko:17,stephan:17,stepl:[17,64],stepr:[17,64],stick:55,sticki:24,still:[2,3,7,9,10,13,17,24,29,32,34,36,37,38,42,44,46,51,53,54,57,58,59,60,64,66,67,74],stm:17,stmaryrd:75,stock:17,stolz:17,stone:54,stop:[3,5,12,17,24,32,38,52,54,57,71],stop_profil:17,store:[17,27,52,53,57,59,60],stori:30,storm:17,str:[0,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],straightforward:[3,55],straightforwardli:3,strat:3,strategi:[7,9,13,17,24,25,26,55,57,59,60,71,77],stratego:[3,77],strategy_level:[64,71],strategy_level_or_var:[64,71],stratif:24,stream:[0,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],stream_eta:30,stream_ext:30,streamlin:[17,24],strength:24,strengthen:[17,35,57,67],strict:[2,5,13,14,17,24,25,31,39,41,42,54,57,58,59,60,66,71],stricter:[13,14,17],strictli:[8,11,14,17,41,57,71],strictprop:[12,17],strikeout:66,string:[2,11,13,14,17,25,29,40,42,51,53,54,55,57,59,64,66,74,75],string_as_ot:17,string_get:36,string_length:36,string_scop:[17,42,71],string_typ:36,stringsyntax:17,strip:[17,58],strong:[17,24,27,31,34,64,67,77],strong_induction_l:17,stronger:[3,12,17,34],strongli:[11,15,17,34,35,44,53,54,57,59],strub:17,struct:[0,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],structur:[2,3,4,8,9,13,17,24,25,27,32,34,35,36,37,38,40,44,45,53,54,58,59,66,67,71,72,77],stt:12,stuck:[12,13,17],studi:[24,31],stuff2:53,stuff:[24,53,75],style:[6,17,24,25,30,37,52,55,57,62,67],suarez:24,sub:[2,4,8,17,27,36,41,46,51,53,54,57,59,60,67,71],sub_equ:72,subcas:[40,75],subclass:[4,10,13,27,39,42,59],subcompon:[17,51],subdir:[17,51,53],subdirectori:[17,27,51,53,59,60],subequ:67,subexpress:[54,58,71],subgoal:[5,11,13,17,24,25,27,54,57,58,60,62,64,67],subgraph:[14,17],subject:[10,17,25,26,30,31,50,51,72],sublemma:17,submak:53,submit:[24,27],submodul:[17,35],subnk:57,subnn:57,subpackag:59,subpart:54,subpattern:[25,54,55],subprocess:17,subproof:[17,34,66,67],subrel:[17,25],subscript:29,subsecond:53,subsect:[17,24,34,42,75],subsequ:[8,14,17,29,37,38,51,54,55,58,59,66,67,71],subsequent_lett:29,subset:[5,9,17,24,25,34,39,44,55,57,58,66,71,77],subset_bi:71,subst:[0,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],substitut:[10,11,17,24,25,26,34,38,46,51,55,57,58,64,67,71],substr:[17,59],substructur:[17,25],subsum:[17,57],subsystem:[17,24],subterm:[3,9,10,11,17,24,25,31,34,41,54,55,57,58,59,64,66,67,71,72],subtim:51,subtitl:75,subtract:[5,57],subtyp:[4,9,14,17,25,31,35,39,77],succ:[2,24,54,59,64],succ_doubl:17,succ_po:17,succe:[2,3,13,17,25,44,46,51,55,57,58,59,60,62,64,66],succeed:[3,17,54,59,72],success:[2,3,4,5,13,17,24,25,34,51,52,55,57,59,60,62,64,66,67,74],successfulli:[13,51,52,54,57,62,63],successor:[24,34,39],succinct:55,suchthat:[6,17],suddenli:55,sudha:17,suff:[17,25],suffic:[52,57],suffici:[3,5,11,13,53],suffix:[3,17,35,51,52,53,54,57,59,71,75],sugar:[2,7,17,28,54,55,59,77],suggest:[11,17,24,25,34,51,52,53,57,66],suit:[2,17,53,57,58,63],suitabl:[17,41,52],sum:[11,17,24,27,35,38,40,55,62,67,71],sum_:[5,7,57],sum_ind:[24,27,71],sum_inequa_rle_lt_depr:17,sum_rec:[27,71],sum_rect:[27,71],sum_sind:[27,71],sumbool:[2,27,46,71],sumbool_ind:27,sumbool_rec:27,sumbool_rect:27,sumbool_sind:27,sumlist:57,summar:[11,51,57,66],summari:[25,46,51,75],summaris:57,summat:57,summer:24,sumor:[27,71],sumor_ind:27,sumor_rec:27,sumor_rect:27,sumor_sind:27,sumxxx:57,sun:24,sunit:12,sunit_rect:12,sup:24,superclass:25,superfici:10,superflu:[17,24],superieur:17,superpos:46,superposit:46,supersed:17,supervis:[17,24],supplement:17,suppli:[17,37,57,62],support:[2,3,4,5,6,8,9,11,13,14,17,24,25,27,30,32,34,35,36,37,40,41,42,44,51,53,54,55,57,59,60,62,63,64,66,71,72,74,75,76],suppos:[3,9,17,51,55,57,64],suppress:[57,75],sure:[2,4,17,35,52,53,58,71],suresn:24,surgic:57,surject:[11,37],surma:17,surpass:17,surpris:58,surround:[3,17,44,57,59,71],survei:[24,25],surviv:[17,24,60,71],suspend:[13,17,66],sustem:59,sven:17,swap:[2,17,54,57,58],swasei:17,sweet:55,sy:53,syllabu:24,sylvain:[17,77],sylvi:24,sym:[3,17,44],sym_equ:[17,57],symbol:[2,3,11,14,17,24,25,27,28,29,31,41,42,43,46,57,59,60,62,64,67,71,75,77],symlink:17,symmetr:[3,17,24,31,59,64,71],symmetri:[3,17,24,34,44,57,60,64],symposium:[24,77],symptom:17,syn_valu:54,sync:17,synchron:[17,24,52],synonym:[17,29,37,51,57,58,64],synopsi:[25,53],syntact:[2,3,11,17,24,25,26,27,28,29,30,31,34,35,37,39,41,57,58,59,64,66,71,74],syntax:[2,4,5,6,8,9,11,13,14,25,26,27,30,32,34,35,37,39,40,41,42,43,45,51,52,53,58,59,60,63,64,66,75,77],syntax_modifi:[17,71],synth:[46,59],synthes:[4,17,24,27,28,42,46,77],synthesi:[17,24,44],synthesis:2,synthesiz:46,synthet:24,system:[3,8,9,11,17,24,25,26,27,28,29,32,33,34,38,39,46,51,52,53,54,55,57,59,60,62,71,73,77],systemat:[17,24,44,55,57,64],t0:57,t1:[3,13,17,34,42,46,57],t2:[17,34,42],t:[0,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,65,66,67,68,69,70,71,72,73,74,75,76,77],t_0:26,t_1:[3,26,31,34,35],t_2:[26,31,34,35],t_:[26,34],t_h:66,t_i:34,t_ind:[17,35],t_k:26,t_m:34,t_n:[3,26,34,66],t_q:34,t_rec:35,t_rect:35,t_scope:[17,71],t_sind:35,t_tauto_intuit:54,tab:[17,29,52,53],tabareau:[3,17,77],tabl:[2,3,4,16,17,24,25,27,35,37,38,46,51,53,54,55,57,59,67,71,75],tableau:24,tableofcont:75,tablog:24,tabul:[17,24,57],tac1:17,tac2:17,tac2alg_constructor:55,tac2def_bodi:55,tac2pat0:55,tac2pat1:55,tac2rec_field:55,tac2rec_fieldexpr:55,tac2rec_fieldpat:55,tac2typ_def:55,tac2typ_knd:55,tac2typ_prm:55,tac:[0,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],tacdef_bodi:54,tacexpr:43,tacl:54,tacmach:17,tacn:71,tactic1:57,tactic:[7,8,9,10,13,16,25,26,29,30,31,32,33,34,35,38,40,41,46,51,52,53,59,62,65,66,73,75],tactic_arg:54,tactic_atom:54,tactic_failur:55,tactic_invoc:58,tactic_list_sep:54,tactic_then_loc:71,tactic_valu:54,tacticm:57,tacticn:57,tacvalu:52,tag:[17,24,51,52,57,66],tail:[17,24,27,46,54,55,57,60,71],tail_add:59,tail_addmul:59,tail_mul:59,tailor:11,taint:51,taiwan:77,takafumi:17,takahashi:77,take:[2,3,5,8,11,12,13,17,24,26,27,28,29,31,32,37,40,41,42,46,51,52,53,54,55,57,58,60,62,64,66,67,71,75],taken:[2,9,13,17,24,34,36,42,44,53,57,64,67,71],talia:17,tame:77,tan:77,tan_atan:17,tan_inj:17,tan_is_inj:17,tanaka:17,tankink:17,tapsoft:24,target:[4,11,17,25,51,58,71],tarski:24,task:[17,57,75],tassi:[8,17,42,57,77],tau:67,tauto:[5,17,24,34,54,62],tauto_gen:54,tauto_intuitionist:54,tautolog:[11,17,24,54,62],taylor:77,tctl:24,teach:17,team:[17,24],tebbi:17,tech_rgt_minu:17,tech_rplu:17,tech_single_z_r_r1_depr:17,technic:[8,17,27,34,44,51,57,71,77],techniqu:[5,9,30,42,57,59,62,67],tediou:[24,34,53,57,67],tej:[17,58],tel:77,telecom:24,telescop:17,tell:[2,3,11,17,24,34,41,42,44,46,51,55,57,60,64,67,71,75],templat:[13,17,25,30,37,40,66],tempor:24,temporari:[2,14,17,24,57],temporarili:[17,53,57,59,66,71],ten:24,tend:[14,57],teo:77,term0:[29,37,55,58,71],term100:[29,40,46],term10:[17,29,32],term1:[28,29,37,44,57],term2:57,term:[2,3,4,9,10,11,12,13,14,17,24,25,27,28,29,30,31,32,33,34,35,36,37,38,39,40,41,42,43,44,46,50,53,57,58,59,60,62,63,66,67,72,75],term_appl:[28,29,37,44,64],term_cast:[29,32],term_cofix:[17,29,30,54],term_evar:[29,43],term_explicit:[29,44],term_fix:[17,29,34,54],term_forall_or_fun:[17,28,29],term_gener:[29,44],term_i:57,term_if:[17,29,46],term_ind:67,term_let:[17,29,32,38],term_ltac:[29,54],term_match:[29,40],term_project:[29,37],term_rec:67,term_record:[29,37],term_rect:67,term_scop:[29,71],term_sind:67,termin:[2,9,17,24,25,27,29,30,32,34,35,38,51,52,55,59,60,66,71,72],terminolog:[24,55],termn:57,termvh:57,ternari:17,terrass:77,territori:52,test:[2,3,4,9,10,11,13,17,24,25,29,30,34,42,46,55,57,58,59,66],test_algebra:42,test_algebraic2:42,test_big_nest:57,test_ind:57,test_sind:57,testbit:[17,59],testbit_div2:17,testbit_eqb:59,testbit_even_succ:17,testbit_fals:59,testbit_nat:59,testbit_odd_succ:17,testbit_spec:59,testbit_tru:59,testcompil:[2,17],tetlei:17,tew:17,tex:[17,53,75],texa:24,texmac:75,text:[17,24,27,51,52,53,57,59,66,71,75],text_:75,textbook:57,textgreek:75,textsf:[0,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],textsl:75,texttt:3,textual:[17,46,71],tgt:53,th:[17,27,30,34,40,57,58,66,67,77],than:[2,3,5,8,11,12,13,14,17,24,29,30,31,34,35,37,43,44,46,51,52,53,54,55,57,58,59,60,62,64,66,67,71,72,73,75],thank:[2,5,12,17,24,34,42,55,57,64,71],the_cmp:42,thei:[2,3,4,6,7,8,9,10,11,12,13,14,15,17,24,25,26,27,28,29,30,31,32,34,35,36,37,38,39,41,42,43,44,45,46,51,52,53,54,55,57,58,59,60,64,66,67,71,72,73,74,75],them:[2,3,9,10,11,13,14,17,24,26,27,28,31,34,35,37,38,40,41,42,43,44,46,51,52,53,54,55,57,58,59,60,62,64,66,67,71,72,73,75],theme:[24,52],themselv:[3,13,14,17,26,35,37,39,41,42,53,57,59,64,71],theorem:[2,5,7,8,11,12,17,24,25,27,29,32,33,35,37,38,42,43,51,52,57,59,60,62,65,66,71,73,74,75,77],theorem_nam:66,theoret:[2,17,24,31,39,77],theori:[3,4,5,11,17,24,25,26,27,28,29,39,42,46,51,53,57,58,60,62,67,71,77],theorylist:17,thereaft:[34,59],therebi:59,therefor:[2,17,29,31,37,52,53,57,58,62,72,73],therein:53,thereof:17,theri:[17,24],thesi:[24,77],thi:[2,3,4,5,6,7,8,9,10,12,13,14,15,17,24,25,26,27,28,29,30,31,32,33,34,35,36,37,38,39,40,41,42,43,44,45,46,50,51,52,53,54,55,57,58,59,60,61,62,63,64,65,66,67,71,72,73,74,75,76],thierri:[17,24,34,77],thing:[17,52,54,55,59,67,72],think:[55,66],third:[2,3,17,25,40,41,44,51,52,53,54,57,58,59,75],thirdli:17,this_scop:57,thisextrafil:53,thm:24,thm_token:[32,59],tho:17,thoma:17,thoroughli:[17,55],those:[2,3,5,10,11,12,17,24,26,33,34,35,37,43,46,52,53,54,55,57,58,59,60,62,64,66,67,71,72],though:[2,8,9,17,24,29,34,35,37,46,51,53,54,55,64,67,71],thought:[9,26,29,63],thread:17,three:[2,4,9,11,17,24,25,34,40,52,53,54,57,59,60,67,71],threeintropatternscombin:58,threshold:[8,17,64,71],throttl:77,through:[3,4,12,17,24,27,28,29,30,32,34,35,36,37,46,52,53,54,55,57,58,59,60,64,65,66,67,71,72,73,74],throughout:[17,29],thrown:2,thu:[2,3,4,5,10,12,17,24,32,34,42,43,46,51,53,54,55,57,58,59,60,64,66,67,71,72,75],thumb:[51,67],thunk:[17,55],ti:[13,57],tie:64,tight:71,timani:17,time1:53,time2:53,time3:53,time:[2,3,5,8,9,11,12,13,14,17,24,25,27,28,29,32,34,36,37,41,42,44,46,52,55,57,58,59,64,66,67,71],time_constr1:54,time_constr:[17,25],time_of_pretty_build_fil:53,timeout:[12,17,25,59,64],timer:54,times_sym:17,timing_fuzz:[17,53],timing_include_mem:[17,53],timing_r:[17,53],timing_sort_bi:[17,53],timing_sort_by_mem:[17,53],timothi:17,timur:17,tip:[17,60],titl:[17,52,75],tj:57,tl:[0,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],tl_map:17,tm:13,tmp:17,tn:[3,13,17,57],to_bit:59,to_bits_of_bit:59,to_constr:55,to_eq:42,to_euclidean_division_equ:[5,17],to_euclidean_division_equations_with:17,to_intro_pattern:17,to_l:42,to_list:17,to_list_append:17,to_list_con:17,to_list_const:17,to_list_exist:17,to_list_fold_left:17,to_list_fold_right:17,to_list_foral:17,to_list_forall2:17,to_list_hd:17,to_list_in:17,to_list_inj:17,to_list_last:17,to_list_map:17,to_list_nil:17,to_list_nil_iff:17,to_list_nth_ord:17,to_list_rev:17,to_list_rev_append:17,to_list_rev_append_tail:17,to_list_tl:17,to_n:17,to_nat:17,to_num_uint:71,to_po:17,to_preterm:17,to_str:[17,55],to_uint:71,to_uint_dec:71,tobia:17,toc:[17,75],todd:75,todo:17,togeth:[2,3,9,17,24,25,27,31,34,35,43,53,54,55,57,66,71,75],toggl:[46,52],toggleabl:17,toi:57,token:[17,29,42,51,52,53,54,55,58,59,66,71,75],toler:17,tolmach:77,tom:17,toni:17,too:[8,9,11,17,54,55,57,58,67,71],took:[17,24],tool:[11,14,25,29,51,52,53,54,57,59,66,71,72,75,77],toolbar:52,toolbox:[3,17],toolchain:[17,51],tooltip:[17,52],top:[3,8,10,12,13,14,17,24,25,27,29,35,37,46,51,52,53,54,55,57,58,59,64,67,71,73,75],top_heap_word:66,topbin:17,topdown:3,topfil:17,toplevel:[2,10,14,17,24,25,27,29,35,44,46,51,52,53,55,57,58,59,60,64,71,72,74],toplevel_selector:[17,29,54,58],toploop:17,toset:[14,17,34],total:[51,53,54],toto:51,toulous:17,toward:[4,17,27,53],tphol:77,trace:[11,13,17,25,32,51,53,57,58,59],track:[17,24,51,53,55,57],tracker:[17,54],tract:77,tractabl:12,tradit:[17,24,51,63],trager:17,traian:17,trail:[17,25,57,74,75],trailer:75,tran:[3,17],trans_equ:57,transact:[64,77],transfer:24,transform:[3,4,11,17,29,57,58,66,67,77],transit:[3,7,8,13,14,17,24,25,26,35,41,44,51,54,57,58,59,60,64,66,74],translat:[2,3,17,24,25,33,41,45,57,71,75],transpar:[3,4,6,9,14,17,24,25,31,32,35,37,41,51,54,55,57,59,60,64,66,67,75],transparentst:17,transport:[12,17],transposit:17,trap:24,travers:[3,17,57,58,67],traverso:77,travi:17,treat:[9,12,13,17,29,46,53,54,57,59,60,62,64,67,71,72],treatment:[2,9,17,40],trece:57,tree:[0,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,68,69,70,71,72,73,74,75,76,77],tree_forest_ind:67,tree_forest_mutind:67,tree_forest_mutrect:67,tree_forest_rec:67,tree_forest_rect:67,tree_ind:[34,67,72],tree_rec:[34,67,72],tree_rect:[34,67,72],tree_sind:[34,67,72],tree_siz:[34,72],tree_size_equ:72,tree_size_ind2:72,tree_size_ind:72,tree_size_rec:72,tree_size_rect:72,treinen:17,tri:[3,4,5,9,13,14,17,34,35,41,46,52,53,54,55,57,58,59,60,62,66,67],triangl:[10,52],triangleright:[26,31],triangleright_:[0,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],trick:[24,55,57,58,72],trickeri:55,tricki:[24,57],trickier:54,trigger:[13,17,25,29,44,54,55,57,60,71],trigonometr:[17,24],trii:[0,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],trili:17,trim:74,trivial:[12,13,14,17,34,46,53,54,55,57,58,60,66,67],trm:54,troubl:[17,54,64,67],true_sub:17,truli:[17,57],trunc:17,truncat:[17,57],trunk:17,trunov:17,trust:[24,33,36,73],truth:[17,54,57],tryif:[17,25],ts:46,tt:[5,13,14,17,27,40,46,54,57],tt_h:66,tt_n:66,tune:[17,38,42,64],tupl:[9,17,37,42,46,55,57,58],turn:[2,8,10,12,13,14,17,24,27,29,32,37,41,42,44,46,51,52,54,55,57,58,59,64,66,67,71],turner:17,tutori:[17,25,63,74,77],tv:2,tweak:17,twice:[17,34,51,59,64,66],two:[2,3,4,5,8,9,10,11,13,14,15,17,24,25,26,27,29,30,31,34,36,37,38,40,41,42,44,46,51,52,53,55,57,58,59,60,63,64,66,67,71,74,75],twofold:28,twoi:57,tx:57,txt:[17,24,53],ty:[54,57],typ:[17,24,34],typabl:[2,4,34],type1:35,type2:35,type:[0,1,5,6,7,8,9,11,12,13,14,15,16,18,19,20,21,22,23,24,25,27,29,31,33,36,39,41,42,43,45,47,48,49,50,51,52,53,56,58,60,61,62,63,64,65,66,68,69,70,72,73,74,75,76,77],type_ind:67,type_of:17,type_rec:67,type_rect:67,type_scop:[13,14,17,25,34,44,46,52,54,58,66,67],type_sind:67,type_term:[17,25],typeabl:3,typecheck:[9,17,41,51,55,58,59,64,66],typeclass:[3,4,5,7,17,25,35,37,38,44,45,58,60,64,66,71],typeclass_constraint:44,typeclass_inst:[13,17,60],typed:[10,55],typeexpand:2,typeset:[17,75],typic:[2,4,6,12,14,17,24,28,29,30,34,35,44,46,51,53,55,57,58,59,60,64,67,71],typo:[17,44],u05d0:17,u0:[10,14,46],u1:[10,13,14,17,57],u2:10,u:[3,4,9,10,14,17,24,26,27,31,34,35,38,39,41,46,53,54,55,57,58,62,64,67,71],u_0:26,u_1:[26,31,34,39],u_2:31,u_:34,u_i:[26,34],u_m:26,u_n:39,ubiquit:57,uconstr:[17,54,71],ui:[17,51],uint63:[17,27,36],uint63_scop:[36,71],uint:[17,59,71],uint_scop:17,uintdecim:71,uinthexadecim:71,uip:[14,17,25,46,59],uip_nil_l:17,uip_nil_nil:17,uip_nil_r:17,uip_none_l:17,uip_none_non:17,uip_none_r:17,uip_refl_nat:67,uj:57,ultim:11,um:[13,57],un:77,unabl:[3,14,34,43,46,53,57,58,59,66,67],unabletounifi:17,unambigu:[17,27,32,44,53,59],unappli:17,unari:[2,3,26,29,34,64],unavail:17,unavoid:57,unbound:[13,14,17,54,55,58],unbox:54,uncapit:17,uncaught:[17,55],unchang:[17,54,57,58,60,64,66],uncheck:59,unclear:[3,10,54],uncom:52,uncommon:17,uncon:17,uncondition:17,uncurri:17,undecid:[29,30],undeclar:[14,17],undefin:[17,28],undelimit:[17,59,71],undeprec:17,under:[5,9,11,17,25,32,40,44,46,52,53,54,55,59,64,66,67],under_rel:17,underli:[9,11,17,24,26,54,57,67,71],underlin:[51,52,66],undermin:57,underscor:[14,17,29,37,44,51,71,75],understand:[3,5,10,12,15,17,24,25,29,33,51,53,54,55,59,60],understood:[17,32,34,36,60,71,75],undertaken:24,undesir:64,undetect:[17,46],undetermin:[57,66],undif:66,undiscrimin:[17,60],undo:[11,17,52,54,58,59,66],undocu:[17,24,59],undon:52,unduli:17,uneed:58,unend:71,unequ:17,uneven:17,unexpect:[17,24,44,53,55,71,73],unexpectedli:54,unfocu:[17,66],unfocus:[17,34,55,59,66,67],unfold:[5,9,13,14,17,24,25,27,31,32,34,37,54,55,57,60,62,66,71],unfold_nth_error:17,unfortun:[3,5,17,42,46,57],unguard:30,unibo:24,unicod:[17,25,75],unicode_id_part:29,unicode_lett:29,unicoq:53,unif:[3,10,13,17,24,25,37,40,42,43,54,60,64,71],unifi:[3,12,13,14,17,34,41,42,43,54,57,58,64,66],uniform:[4,17,24,34,40,44,54,55],uniformli:[17,24,51],uninform:17,uninstal:[17,25],uninstanti:[43,44,54,58,67],unintend:57,unintendedli:17,uninterest:57,uninterpret:[17,62],uninterrupt:17,union:[3,13,17,54,59,66,77],union_compat:3,union_mor:3,uniqu:[2,3,12,13,17,24,27,31,35,38,57,59,67,71],unit:[2,12,13,14,17,27,34,40,46,53,54,55,57,62,64,71],unit_eqdec:13,unit_ind:27,unit_monoid:14,unit_rec:27,unit_rect:27,unit_sind:27,uniti:11,univ:17,univ_annot:[10,14,29,37],univ_constraint:14,univ_decl:[10,14,28,35],univ_level_or_qu:14,univ_name_list:59,unival:17,univers:[3,4,8,9,12,13,17,24,25,26,27,28,29,30,31,32,33,34,37,39,40,44,46,51,54,57,59,62,66,67,71,77],universe_expr:39,universe_nam:[14,39],unix:[17,24],unjustifi:17,unkei:57,unknown:[17,29,42,43,58,60,66,71],unless:[2,3,13,14,17,29,40,41,42,44,51,52,57,58,64,71,72,75],unlik:[10,13,17,24,30,39,52,54,55,57,58,59,60,64,67,71],unload:17,unlock:25,unmaintain:17,unmatch:58,unmodifi:52,unnam:[17,44,52,57,66,71],unnamed_coqscript_:52,unnamed_thm:66,unnatur:71,unnecessari:[8,17,57,62,66],unneed:[8,17,58],unop:5,unopspec:[5,17],unord:[3,17,57],unpack:17,unpredict:54,unprefix:3,unprocess:52,unprotect:[17,57],unprov:[17,43,58],unproven:[52,58,66],unqualifi:[17,35,55,71],unquot:[17,53,55],unquoted_str:53,unread:[17,59],unrealist:24,unreli:17,unresolv:[9,13,17,57,58,60,64,67],unrespons:17,unsaf:[2,17,55,66],unsafe_:17,unsafe_type_of:17,unsafecoerc:17,unsatisfi:[5,60],unselect:58,unset:[4,5,12,14,17,24,25,34,35,37,38,42,44,46,51,54,55,57,59,66,67,71],unshelv:[17,43,66],unsign:[5,17,36],unsolv:[9,17,43,66],unsound:[17,34],unspecifi:[4,14,17,43,55,62,67],unstabl:[14,17],unsuit:8,unsupport:[17,29,35,38,52,59],untermin:71,until:[13,14,17,24,26,31,32,34,40,52,54,55,57,60,64,66,67,72],untouch:[17,41],untyp:[10,17,25,55,71],unus:[17,25,53,58,71],unusu:17,unwant:17,up:[3,8,13,17,24,25,26,31,34,35,38,42,43,52,53,54,55,57,58,64,66,67,71,75],upcom:17,updat:[4,8,15,17,24,36,37,46,52,53,58,59,67,71],upfront:53,upgrad:[15,17,25],upon:[5,11,36,43,51],upper:[10,14,17,39,44,52],upper_bound_thm:17,uppercas:[29,55],upstream:[17,53],upward:[17,24],url:[17,27,52,75,77],us:[2,3,5,6,7,8,9,10,11,12,13,17,24,26,27,28,29,30,31,32,33,34,36,39,40,41,42,45,55,57,59,60,61,62,63,65,72,73,74,75,77],usa:77,usabl:[2,17,24,38,52,66,67,71],usag:[17,24,25,27,51,53,54,58,60,64],usecamlp4:17,usefulli:17,useless:[13,14,17,24,25,37,46,60],uselessli:17,uselocaldef:17,usepackag:75,user:[4,5,6,7,8,9,11,12,13,14,17,25,29,32,33,34,35,36,37,39,42,43,44,45,46,51,52,53,54,55,57,58,59,61,62,64,65,66,67,71,72,73,74,75,76,77],usernam:52,usual:[3,8,9,12,17,25,26,27,28,30,34,35,37,40,43,44,46,52,53,54,55,57,58,59,60,62,64,66,67,71,74,75],utf8:[52,53,75],utf8x:75,utf:[17,52,75],util:[17,42,51,53],v1:[25,50,57],v2:[24,57],v3:[24,57],v4:24,v5:24,v6:24,v7:[17,24],v8:17,v:[2,3,7,8,11,12,14,17,24,26,27,34,35,37,42,44,46,51,52,53,54,55,57,58,59,67,71,75],v_0:11,v_1:[11,31],v_2:11,v_3:11,v_:[11,26],v_i:[11,31],v_m:31,vadim:17,val:[2,34,55,57],valentin:17,valid:[2,3,4,5,8,10,11,14,17,25,26,29,32,34,35,40,42,51,54,55,57,58,59,66,71,72],valu:[2,4,5,6,9,11,12,13,14,17,24,25,26,27,28,29,31,32,34,36,37,38,40,42,43,51,52,53,57,58,59,60,62,64,66,67,71,74],value_tact:[52,54,64],van:17,vanish:24,vari:[24,54,58,67,71],variabl:[2,3,4,5,6,7,8,9,10,12,13,14,17,24,25,26,27,28,29,31,32,34,35,37,38,39,40,41,42,45,53,54,57,58,59,60,62,64,67,71,72,75],varianc:[3,17],variant:[5,13,14,17,24,25,27,28,29,32,33,34,35,37,38,42,51,54,55,59,60,63,64,66,67,71,72],variat:[17,59,77],varieti:[17,24],variou:[3,16,17,24,25,27,28,29,34,44,51,52,53,55,57,58,59,60,64,66,71],varmap:5,varnam:37,varner:17,varref:55,vassor:17,vax:24,vbt98:[3,77],vcon:[17,67],vdash:[0,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],vdfile:17,ve:[17,52,53,66,67],vec:67,vec_ind:67,vec_rec:67,vec_rect:67,vec_sind:67,vector:[17,46,67,71],vector_ind:67,vector_rec:67,vector_rect:67,vector_scop:17,vector_sind:67,vectordef:17,vectornot:17,vectorspec:17,vener:17,verbatim:25,verbos:[13,17,42,51,59],veri:[2,8,9,11,13,17,24,25,27,29,34,42,46,52,53,54,55,57,58,59,60,62,64,66,67],verif:[3,24,25,32,66,67,77],verifi:[3,7,9,11,14,17,24,25,29,31,32,33,35,51,60,66],verlag:77,vermand:17,vernac:[17,24,51,53,71,75],vernac_control:71,vernacular:[17,24,35,38,59,63,75],version:[2,3,4,7,9,13,14,15,25,29,32,34,35,36,37,41,46,50,51,52,57,58,59,60,62,66,73,74,75,77],versu:67,vertic:[17,59,71],vfile:53,vi:53,via:[2,5,8,11,17,35,51,53,54,55,57,59,71,72],vicent:17,view:[2,11,17,25,26,29,32,34,39,41,52,55,60,66],vincent:17,vindum:17,vio2vo:17,vio:17,violat:[39,66],virtu:17,virtual:[17,24,32,53,64],vis01:[3,77],visibl:[6,17,24,38,52,57,60,66,71,75],visser:[3,77],visual:[17,51,52,54,66,71],vlad:72,vm:[10,17,58,59,64],vm_c:53,vm_cast_no_check:58,vm_comput:[5,17,25,32,36,51,58],vmbyteflag:17,vnil:67,vo:[8,17,24,25,53,59],vocabulari:25,vofil:53,vok:[17,51],volatil:[17,32,41,46],volum:[24,77],volunt:17,vote:24,vs:[13,17,25,26],vscoq:[8,17,51,53,66],vulner:17,w:[0,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],w_1:[26,31],w_i:26,w_m:[26,31],wa:[2,3,10,11,12,17,24,27,28,29,32,34,35,37,38,41,42,43,44,51,52,53,54,55,57,58,59,60,63,64,66,67,71,72],wai:[2,3,5,11,12,13,14,17,24,25,26,27,29,30,31,32,34,35,37,42,43,44,46,51,52,53,57,58,59,60,62,63,64,66,67,71,72,73,75],wait:[17,55,66],waitpid:17,walding:24,walk:[55,71],wall:64,wand:77,wang:17,want:[2,11,13,17,34,35,36,41,42,43,51,52,53,54,55,57,58,59,60,62,64,66,67,71,73,74],warn:[2,3,4,10,12,13,16,17,24,25,27,28,29,32,34,35,37,41,42,44,46,51,52,54,55,57,59,60,62,66,71,72],we:[2,3,4,5,9,11,12,13,14,16,17,24,26,27,28,29,30,31,33,34,35,38,39,40,42,44,45,46,51,52,53,54,55,57,58,59,60,64,66,67,71,72,75],weak:[5,17,25,27,35,55,64,67,71],weaken:[17,67],weaker:[3,17,24,60],weakli:64,web:[17,27,52,53],websit:[17,75,76],wedg:7,weegen:17,week:17,wei:24,weid:17,weight:17,weird:17,welcom:[17,54],well:[2,3,4,8,9,10,11,13,14,17,24,25,26,29,30,31,32,33,35,37,39,43,45,46,51,52,53,54,55,57,58,59,63,64,66,67,71,72,74,75],well_found:27,well_founded_ind:27,well_founded_induct:[17,27],wellfound:[9,17,27],wendl:17,weng:17,went:[17,54,55],wenzel:17,wer94:[31,77],were:[3,11,13,17,24,34,35,36,38,42,44,51,53,54,55,59,60,66,71,72,75],werner:[11,17,24,77],wev:[0,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],weval:35,wevt:[0,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],weyhrauch:24,wf:[0,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],wf_lex_exp:17,wf_nat:[2,17,24],wf_simul:17,wf_slexprod:17,wf_z:24,wfe:[0,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],wft:[0,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],wftwolin:[0,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],what:[2,3,5,10,13,16,17,24,25,27,29,33,34,35,41,42,46,51,53,54,55,57,59,60,64,66,67,71],whatev:[3,44,64,75],whelp:17,when:[2,3,4,5,6,7,8,9,10,11,12,13,14,15,17,24,25,27,28,29,30,32,34,35,36,37,38,39,40,41,42,43,45,51,52,53,54,55,58,59,60,62,64,66,67,71,72,74,75],whenev:[3,7,14,17,27,29,42,55,57,62,64,67,71],where:[2,3,4,5,6,7,8,9,10,11,12,13,14,17,24,26,27,29,30,34,35,36,37,38,40,41,42,43,44,46,51,52,53,54,55,57,58,59,60,62,64,66,67,71,72,75],wherea:[17,29,54,55,57,58,62,74],wherev:[31,53,54,67,71],whether:[2,3,9,10,12,13,14,17,29,34,35,41,44,51,52,53,54,55,57,59,62,64,66,71,75],which:[2,3,4,5,6,7,8,9,10,11,12,13,14,17,24,25,26,27,28,29,30,31,32,33,34,35,36,37,38,39,40,41,42,43,44,45,46,51,52,53,54,55,57,58,59,60,62,63,64,65,66,67,71,72,73,75],whichev:17,whilst:9,white:[17,57],whitequark:17,whitespac:[17,24,53,75],who:[17,24,54,57,59],whole:[2,3,9,11,17,29,40,46,51,52,53,55,57,59,71,75],whose:[2,3,4,5,11,13,14,17,24,26,27,30,31,33,34,35,37,39,41,42,44,46,53,54,55,57,58,59,60,64,67,71,75],why2:17,why3:17,why:[3,11,17,34,37,43,55],wide:[29,38,52,53,58],widget:24,width:[17,59,71],wiedemann:17,wiedijk:24,wiki:[17,64],wikipedia:64,wilcox:17,wild:[17,57],wildcard:[9,13,25,28],william:77,win:17,window:[8,17,24,51,52,53],winterhalt:[17,77],wire:[17,55],wish:[2,5,17,53],wit:[5,14,17,24,27,39,55,64],with_declar:[17,35],with_strategi:[17,64,71],with_uniform_flag:54,within:[5,17,24,28,29,31,33,35,37,38,41,42,44,51,52,54,55,58,59,60,64,66,71],without:[2,3,5,8,9,11,13,14,17,24,26,29,32,33,34,35,37,42,43,44,46,51,52,53,54,55,57,58,59,60,63,64,66,67,71,74,75,77],wizard:14,wlia:5,wlog:[17,25],wlog_stat:57,wlra:5,wlra_q:5,wml07:77,wnia:5,wnra:5,wojciech:17,wolf:17,won:[17,25,38,52,53,54,55,58,62,64,67,71,73],word:[4,14,17,27,30,42,51,52,53,55,58,66],work:[2,3,4,5,9,10,12,13,17,24,25,26,27,32,35,41,42,43,46,51,52,54,55,57,58,59,64,67,71,74,77],workaround:[53,54,55,60],worker:[8,17,52,54],workflow:17,workshop:[24,77],workspac:17,workstat:24,world:[12,17,24,55,57,77],wors:55,worst:[17,59],worth:57,would:[2,3,4,11,14,17,28,29,30,31,32,34,37,41,42,43,44,46,53,54,55,57,58,59,60,62,64,66,67,71,72,75],wpsatz:5,wrap:[9,12,13,17,36,38,53],wrapper:[17,53,67,71,72],write:[3,4,8,11,13,14,17,24,25,26,27,29,31,32,33,34,38,39,43,51,53,54,55,57,58,59,63,66,67,71,73,75],writer:[17,29,55],written:[2,3,5,11,13,17,24,26,28,29,34,35,36,37,42,43,44,46,52,53,54,55,57,59,64,71,73,74],wrong:[2,3,17,24,44,51,54,66,72],wrongli:[17,46],wrongplu:34,wrote:[11,17,24],wrt:[17,24],ws:[0,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],wse:[0,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],wsl:52,wso:5,wt:[0,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],wte:[0,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],wteg:[0,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],wtm:[0,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],www:[17,24,25,27,50,75,77],x0:[3,13,17,37,43,44,54,66,71],x1:[3,9,13,17,27,42,54,57,59,60,72],x1p:36,x2:[3,27,42,59,60,72],x3:[27,71,72],x3p1:71,x3p2:71,x:[0,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],x_1:[7,26,34,35],x_:[7,34],x_j:34,x_k:[26,34],x_m:34,x_n:7,xa:57,xarg:17,xavier:[17,77],xb:57,xcolor:75,xdg:[17,53],xdg_config_hom:[17,51,52],xdg_data_dir:[17,51],xdg_data_hom:[17,51,53],xi:17,xia:17,xl:57,xlia:5,xlra:5,xmailserv:77,xml:[17,24],xn:[3,9,17,57],xnia:5,xnra:5,xo:17,xor:17,xorb:[17,27,59,62],xorb_comm:59,xp:17,xpsatz:5,xs:[58,64,67],xso:5,xx:17,xxx:14,xxx_scope:17,xxy:11,xyz:17,xz:11,y0:[3,13,43],y13:66,y1:[13,27,42,46,59],y2:[27,42,59],y3:27,y:[2,3,4,5,9,11,12,13,14,17,24,26,27,28,31,34,35,36,37,38,40,41,42,43,44,46,52,54,55,57,58,59,60,62,64,66,67,71,77],y_1:[34,38],y_:34,y_gt1:57,y_j:34,y_lt2:57,y_lt3:57,y_m:34,y_n:38,yale:17,yang:17,yann:[17,24],yannick:17,yao:17,ybertot:17,ye:[4,9,11,14,17,29,34,37,42,51,53,59,67],year:[17,24],yellow:[17,52],yet:[2,17,42,43,46,51,52,54,55,57,58,60,66,71,72],yice:17,yield:[4,11,17,24,31,46,54,55,58,67,71],yishuai:17,ym:57,ymmv:17,yojson:53,yop:24,york:77,yoshihiro:17,you:[2,3,4,7,8,10,11,13,14,15,16,17,24,25,27,29,32,34,35,37,41,43,44,46,51,52,53,54,55,57,58,59,60,62,64,66,67,71,72,73,74,75],your:[2,3,8,11,14,15,17,25,29,51,52,54,55,57,58,59,60,62,66,71,73,74,75],ype:77,ys:[46,58,67],ystem:77,yusuk:17,yve:[17,24,72],yx:11,yyy_scop:17,yz:11,z0:[11,17,71],z2nat:17,z3:17,z:[3,5,7,11,13,14,17,24,26,27,28,29,34,35,37,40,41,42,44,54,55,57,58,59,60,64,66,67,71],z_div_mod_eq:17,z_div_mod_eq_ful:17,z_le_gt_dec:17,z_lt_induct:17,z_lt_le_dec:17,z_scope:[5,11,17,27,66,71],za:[17,71],zaliva:17,zar:17,zarith:[5,11,17,24,27,29,53,57,60,66],zarith_aux:17,zarith_bas:17,zarith_base_modul:17,zarithr:11,zbinari:17,zbitwis:17,zchines:24,zcomplement:[17,24],zdigit:17,zdiv:17,zdiv_eucl_po:17,zdiv_fact:17,zdiveucl:17,zeimer:17,zeldovich:17,zenon:17,zero:[3,7,11,17,26,27,37,42,46,53,54,55,58,59,60,64],zeroon:[0,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],zeta:[17,24,31,55,64],zeuclid:17,zfc:24,zgt_square_simpl:17,zhong:77,zifi:[17,25],zify_convert_to_euclidean_division_equations_flag:5,zify_plugin:[11,27,29,36,54,55,57,60,66],zify_post_hook:[5,17],zify_pre_hook:[5,17],zifybool:[5,17],zifyclass:[5,17,57],zifycomparison:5,zifyinst:5,zifyint63:17,zifyn:[5,17],zifynat:[5,17],zifypow:17,zifysint63:5,zifyuint63:5,ziliani:[17,77],zim19:[74,77],zimmerman:[17,24],zimmermann:[17,77],zinc:[17,64,77],zine:77,zle:17,zle_0_plu:17,zle_mult_simpl:17,zle_zmult_pos_right:17,zle_zmult_right2:17,zlogarithm:[17,24],zlt_gt_succ:17,zlt_square_simpl:17,zlt_succ_gt:17,zmax:17,zmin:17,zminmax:17,zmisc:17,zmod:17,zmod_mod:17,zmod_neg_bound:17,zmod_pos_bound:17,zmodulo:17,zmult:24,zmult_1_n:17,zmult_assoc:17,zmult_assoc_l:17,zmult_comm:11,zmult_le_compat_r:17,zmult_minus_distr:17,zmult_on:17,zmult_zminus_distr_l:17,zmult_zminus_distr_r:17,zn2z:17,znatpair:17,znumtheori:17,zodiv:17,zplu:17,zplus_assoc:17,zplus_assoc_l:17,zplus_comm:17,zpo:17,zpower:[17,24],zpred:17,zsgn:24,zsqrt_compat:17,zulip:[17,52,54],zwanenburg:24,zx:11,zy:11,zyuzin:17},titles:["<no title>","<no title>","Program extraction","Generalized rewriting","Implicit Coercions","Micromega: solvers for arithmetic goals over ordered rings","Program derivation","Nsatz: a solver for equalities in integral domains","Asynchronous and Parallel Proof Processing","Program","User-defined rewrite rules","ring and field: solvers for polynomial and rational equations","SProp (proof irrelevant propositions)","Typeclasses","Polymorphic Universes","History and recent changes","Indexes","Recent changes","Attribute index","Command index","Errors and warnings index","Flags, options and tables index","Tactic index","General index","Early history of Coq","Introduction and Contents","Typing rules","The Coq library","Functions and assumptions","Basic notions and conventions","Coinductive types and corecursive functions","Conversion rules","Definitions","Core language","Inductive types and recursive functions","The Module System","Primitive objects","Record types","Sections","Sorts","Variants and the match construct","Setting properties of a function's arguments","Canonical Structures","Existential variables","Implicit arguments","Language extensions","Extended pattern matching","<no title>","<no title>","<no title>","<no title>","The Rocq Prover commands","CoqIDE","Building Rocq Projects","Ltac","Ltac2","<no title>","The SSReflect proof language","Tactics","Commands","Programmable proof search","Automatic solvers and programmable tactics","Solvers for logic and equality","Creating new tactics","Reasoning with equalities","Basic proof writing","Proof mode","Reasoning with inductive types","<no title>","Glossary index","<no title>","Syntax extensions and notation scopes","Functional induction","Libraries and plugins","Writing Rocq libraries and plugins","Documenting Rocq files with coqdoc","Command-line and graphical tools","Bibliography"],titleterms:{"0":[17,24],"0beta":17,"1":[17,24,37,67],"10":17,"11":17,"12":17,"13":17,"14":17,"15":17,"16":17,"17":17,"18":17,"19":17,"1beta":17,"1gamma":17,"2":[17,24,37,67],"20":17,"3":[17,24,71],"4":[17,24],"4beta":17,"4beta2":17,"5":[17,24],"5beta1":17,"5beta2":17,"5beta3":17,"5pl1":17,"5pl2":17,"5pl3":17,"6":[17,24],"6beta1":17,"7":[17,24],"8":17,"9":17,"\u03b1":31,"\u03b2":31,"\u03b4":31,"\u03b6":31,"\u03b7":31,"\u03b9":31,"abstract":[57,66],"boolean":[46,54,57],"byte":36,"case":[5,24,40,52,57,58,67],"catch":[54,55],"class":[3,4,37,55,71],"default":[41,46],"do":[11,54],"float":[27,36],"function":[4,28,30,34,41,44,54,60,72],"long":24,"new":[3,11,17,24,35,53,57,63],"short":5,"static":55,"switch":[55,57],"try":54,A:[2,14,35,58,67],In:55,Is:11,No:53,One:57,The:[11,26,27,34,35,44,51,53,57,71,75],_coqproject:53,abbrevi:[55,57,71],about:[7,46,71],access:37,ackermann:60,acknowledg:57,activ:4,ad:[3,11,52],addit:[2,57,60],advanc:[57,72],algorithm:64,alia:74,alias:46,altern:[41,54],alwai:64,ambigu:3,an:[35,57,59,67],analysi:67,annot:8,anonym:[37,57],antiquot:55,api:55,appendix:25,appli:[43,57,58,64,67],applic:[4,28,44,54,58],ar:[57,66],argument:[2,37,41,44,46,53,57,67,71],arithmet:[5,27],ariti:34,arrai:36,ask:9,assert:32,assert_fail:54,assert_succe:54,assign:57,associ:71,assumpt:[28,57],asynchron:[8,52],attribut:[4,17,18,29,35,38],autom:60,automat:[8,11,34,41,43,44,61,67],avail:4,avoid:2,axiom:2,b:58,backtrac:54,backtrack:[54,55,59],backward:[3,58],base:36,basic:[12,27,29,52,53,54,57,65,71],batch:51,beta1:17,beta2:17,beta3:17,beta:31,between:[2,55,59,66],bibliographi:77,bidirection:41,bind:[13,41,52,55,58,71],binder:[3,28,44,57,71],block:[8,57],bookkeep:57,both:71,bound:71,brace:66,branch:[54,57],breakpoint:52,buffer:52,build:[13,53],built:55,bullet:[57,66],calcul:66,calculu:26,call:[52,55],can:43,canon:42,cast:32,casual:44,caveat:[8,30],cell:55,chain:57,chang:[15,17,24,55],charact:52,check:54,checker:51,classic:58,claus:[37,46,58],clear:57,co:30,code:2,coercion:[4,46,71],cofix:30,coinduct:30,combin:[44,58,67],command:[3,13,17,19,24,35,51,52,57,59,66,67,71,75,76],comment:53,common:[53,58],compact:42,comparison:[54,55],compat:[10,17,37,55,57,74],compil:[17,51,52,53,59],complex:71,compon:55,compound:58,comput:[53,54,64],conclus:59,concret:[11,24],condit:[34,54,57],configur:53,conflict:2,confluenc:10,congruenc:57,connect:27,constant:[3,37,59,71],constraint:[14,66],construct:[12,24,26,34,37,40,54,59],constructor:[34,67],content:25,context:[3,13,54,55,57,58],contextu:[44,57],continu:[3,41,44],contradict:58,contravari:3,contribut:[2,24,27],control:[9,35,44,46,54,57,58,59,64,66],convent:[29,46],convers:[14,31,64],convert:31,coq:[24,27,52],coq_makefil:53,coqc:[51,53],coqchk:51,coqdep:53,coqdoc:75,coqid:[17,52],coqmakefil:53,coqrc:51,coqtop:51,core:33,corecurs:30,correct:34,count:54,covari:3,creat:[35,37,43,60,63],cumul:14,curli:66,custom:[51,52,71],cut:[5,54],cycl:66,databas:60,datatyp:27,deactiv:44,deal:11,debug:[12,54,55,59],debugg:[52,54],decid:[54,67],decis:5,declar:[3,13,38,41,42,44,55,57,66,67],defect:[54,57],defin:[10,34,35,37,54,55,60],definit:[3,9,12,14,30,32,34,37,40,46,54,55,57,64,71],delai:[55,66],delta:31,demonstr:14,depend:[17,46,53,58,59,67],deprec:[3,74],deriv:[6,42,67],descript:5,design:55,destruct:67,destructor:34,destructur:[46,57],detail:[2,17,24,53],detect:54,diff:66,differ:[2,44,66],disabl:71,disambigu:59,discharg:57,discrimin:67,discuss:11,disjunct:46,displai:[4,43,44,52,59,71],divis:2,document:[29,53,75],doe:[11,46],doesn:64,domain:7,dune:53,dynam:55,e:43,eappli:43,earli:24,eauto:13,edit:52,effect:[41,55],effici:24,elabor:9,element:[54,58],elim:57,elimin:[2,46,57],embed:53,emphasi:75,enabl:[3,66,71],encod:[12,52],end:[34,38],enter:66,entri:[57,71],environ:[51,59],equal:[7,9,27,62,64,67],equat:[11,57],equival:[57,58],error:[8,20,54,55],escap:75,essenti:29,eta:10,euclidean:2,eval:[54,64],evalu:[54,55],even:67,exact:57,exactly_onc:54,exampl:[2,3,4,5,6,11,14,17,26,27,28,29,30,31,34,35,37,38,40,41,42,43,44,46,51,52,53,54,55,57,58,59,60,62,64,66,67,71,72,74,75],except:55,execut:54,exist:[2,24,35],existenti:[43,57],exit:66,expans:[31,46],explicit:[14,43,44,57],explicitli:44,expos:59,express:[46,54,55,71],extend:[46,57],extens:[3,24,45,46,57,71],extra:[2,59],extract:[2,17,24],factor:[46,71],fail:[46,54,57],failur:54,famili:57,fast:[59,64],fatal:55,ffi:2,field:[11,35,37],file:[51,52,53,59,74,75],filenam:[2,53],fill:54,first:[3,34,46,54,57],fix:[31,34],fixpoint:[9,34],flag:[17,21,29,59],flow:[54,57,58],focus:[54,66],fold:64,fold_right:64,follow:44,foral:28,forbidden:53,forest:67,form:34,forward:58,found:27,frequent:9,fresh:54,from:[35,44,55],full:59,fun:28,function_scop:71,functor:35,gallina:57,gener:[2,3,4,11,14,23,29,44,54,55,57,67,71,72],get:[54,57],give:44,given:34,global:[14,54,71],glossari:69,goal:[5,11,54,55,57,58,66,67],grammar:[24,53],graph:4,graphic:76,guard:54,hand:46,have:[54,57],helper:67,hidden:46,hide:75,hierarchi:[13,42],high:5,higher:10,hint:[41,57,59,60],histor:24,histori:[11,15,24],hole:[10,54],horror:2,how:[11,66],html:75,hyperlink:75,hypothes:[54,55,58,59,66],hypothesi:[54,58],ident:[4,54],identifi:[59,71],idtac:54,implicit:[4,41,44,46,60,71],implicits_alt:41,impred:26,includ:58,incompat:[3,17],indent:57,index:[16,18,19,20,21,22,23,34,57,69],induct:[2,26,34,40,46,67,71,72],infer:[17,43,44],infix:71,inform:[66,71],infrastructur:17,inherit:[4,71],inlin:[2,59],innermost:3,input:52,insert:44,insid:[53,54,75],instal:53,instanc:[13,43],integ:[5,27,36,71],integr:7,interact:[8,35,44,51,54,55,57],interdepend:53,interfac:51,intern:59,interpret:[57,71],intro:[57,58],introduc:74,introduct:[3,25,57],intuitionist:54,invers:67,inversion_sigma:67,invoc:58,involv:[46,71],io:55,irrefut:46,irrelev:[12,31],is_cofix:54,is_fix:54,is_proj:54,isomorph:54,issu:[12,17,57],item:[35,57],iter:57,j:53,kei:52,kernel:17,keyword:[58,59],kind:44,knowledg:44,languag:[2,17,24,25,33,45,55,57],larger:67,late:53,latex:[53,75],launch:51,law:10,layer:55,lazy_match:55,lazymatch:54,least:54,left:67,leibniz:64,lemma:[9,27,66],let:[24,32,46,54,57],level:[5,10,29,30,32,34,55],lexic:29,lia:5,librari:[17,24,27,51,53,59,60,71,73,74],licit:57,limit:67,line:[17,51,75,76],linear:5,liner:57,list:[27,54,55,75],load:[51,53,59],local:[14,29,35,38,46,53,54,57,58,60,71],locat:[59,71],lock:57,logic:[27,53,54,60,62],loop:54,low:55,lower:34,lra:5,ltac1:55,ltac2:[17,55],ltac:[17,54,55],maccarthi:60,machin:59,macro:54,main:24,mainten:66,make:54,man:53,manag:[52,58,66],manipul:54,manual:[17,41,44],map:11,match:[31,34,37,40,46,54,55,57],materi:75,maxim:44,mechan:57,memori:66,meta:55,metavari:57,micromega:5,minim:14,miscellan:[17,24],ml:[2,55],mode:[8,44,52,55,57,66],modifi:53,modul:[4,35,53],monomorph:14,more:7,morphism:3,move:[57,58],multi:57,multi_match:55,multimatch:54,multipl:[37,41,46,53,54,55,57],museum:2,must:46,mutabl:55,mutual:34,n:67,name:[24,35,37,54,66],nat:[27,29],nativ:[17,53],native_comput:[53,64],natur:[54,55,60,67],neg:34,nest:[34,46],nia:5,non:[5,12,34,44,54,55,58,67,71],noncumul:14,nonreflex:3,nonsymmetr:3,notat:[17,27,42,54,55,59,71],notion:29,novelti:24,nra:5,nsatz:7,number:[27,54,60,71],numgoal:54,object:[34,36,46,74],oblig:9,ocaml:59,occurr:[34,57,58,67],odd:67,old:17,omit:35,onc:54,opam:53,opaqu:13,open:71,oper:59,optim:[2,54],option:[2,17,21,29,51,66,75],or_and_intropattern:67,order:[5,10,58],orient:58,other:[17,44,66],outermost:3,over:[5,9,55,57],overflow:29,overload:42,overview:[53,55],own:53,packag:53,page:53,parallel:8,paramet:[35,46,51,57],parameter:[13,34,71],parametr:[3,46,57],pars:[24,44,55,71],part:[59,75],partial:58,path:[53,59],pattern:[10,44,46,54,55,57,58,59,71],peano:27,perform:[53,58],permut:54,phrase:53,plane:5,plugin:[73,74],polymorph:[10,14,34,57],polynomi:11,posit:34,positivstellensatz:5,potenti:17,pre:5,preced:71,precompil:53,predefin:71,predic:[46,57,67],prefer:52,prelud:27,premis:[58,67],present:[4,14],preserv:10,pretti:[43,44,46,75],primit:[27,36,37,59,71],principl:[67,72,75],print:[3,4,14,37,43,44,46,54,55,59,71,75],privat:40,procedur:5,process:[5,8,54],produc:51,product:58,profil:[51,54,55],program:[2,6,9,27,55,60],programm:[60,61],progress:54,project:[37,53],proof:[5,8,12,14,25,31,32,46,54,57,58,60,65,66],prop:34,properti:[41,54,71],proposit:[12,27,54],prove:[54,66,67],prover:[25,51,53],provid:[3,46],psatz:5,qualifi:35,quantifi:27,queri:[52,59],question:9,quit:59,quot:53,quotat:55,radix:71,ration:[5,11],real:[5,17,27],realiz:2,reason:[58,64,67],recent:[15,17],record:[4,37],recurr:57,recurs:[27,30,34,55,71,72],redex:57,reduct:[24,31,34,37,55,59,64],refer:[17,54,59],reflect:57,refut:5,regist:59,registr:59,relat:3,remark:57,renam:41,reorder:[54,66],repeat:54,repetit:57,request:[59,66],reserv:[58,71],resili:8,resolut:[43,44,57],reus:37,revers:[4,44,54,55,64],revgoal:66,rewrit:[3,10,57,64,67],right:[46,67],ring:[5,11],rocq:[2,25,51,53,57,60,71,74,75],root:[24,53],rule:[10,26,31,34,38,57,64,71,75],run:[52,54],s:[2,27,41,67],same:[46,53],save:52,scheme:[67,72],scheme_typ:67,scope:[35,41,71],script:[51,52],search:[59,60],searchpattern:59,searchrewrit:59,second:[34,46,54,58],section:[4,13,14,38,66,75],select:57,selector:[54,57],semant:55,separ:66,sequenc:54,set:[2,13,26,29,37,41,57,58,60,66],setoid:[3,64],setup:53,share:35,shelv:66,shelve_unifi:66,shortcut:57,show:[66,75],side:[11,46],simpl:[28,31,34,35,55,64,71],simple_bind:58,simplif:57,simultan:71,singl:[51,54],soft:54,solv:[9,43,54,66],solver:[5,7,11,61,62],some:[2,27,35],sort:[14,34,39],sourc:[17,75],special:[57,58],specif:[17,25,27],specifi:14,split:[5,53],sprop:12,ssreflect:[17,57],stack:[29,52],standard:[17,24,27,55,57,60,71],start:[51,57],state:66,statu:59,step:[57,66],strategi:[3,46,64],strict:[12,34,44,55],strictli:34,string:[27,36,71],structur:[11,42,57],style:75,sub:35,subgoal:66,subpattern:46,subrel:3,subset:53,substitut:54,substructur:13,subterm:[43,46],subtyp:[26,44],succe:54,success:54,suff:57,suggest:8,summari:[13,17,24,35,38],superclass:13,support:[10,29,52],survei:27,swap:66,symbol:[10,52,54],synopsi:57,syntact:[9,54,55],syntax:[3,10,17,24,29,44,46,54,55,57,71],system:[2,35],t:64,tabl:[21,29],tactic:[3,5,11,17,22,24,27,43,54,55,57,58,60,61,63,64,67,71,72,74],target:[2,53],templat:[34,52],term:[26,54,55,64,71],termin:[10,12,57],test:[53,54],theorem:58,theori:34,thi:11,time:[51,53,54],time_constr:54,timeout:54,tool:[17,24,76],top:[30,32,34],toplevel:54,trace:54,trail:44,transit:55,transpar:13,tree:67,trigger:74,tryif:54,two:[35,54],type:[2,3,4,10,17,26,28,30,32,34,35,37,38,40,44,46,54,55,57,59,67,71],type_scop:71,type_term:54,typeclass:[13,57],uip:12,under:[3,57],understand:46,undo:64,unfold:[3,41,64],unicod:52,unif:[14,58,66],uninstal:53,univers:[10,14],unlock:57,unreleas:17,unset:29,until:58,untyp:54,unus:46,up:51,upgrad:53,us:[4,14,25,35,37,38,43,44,46,51,52,53,54,58,64,66,67,71],usag:[3,11,57,66,75],useless:2,user:[2,3,10,24,27],valu:[3,46,54,55],variabl:[11,43,44,46,51,52,55,66],varianc:14,variant:[40,46,57,58],variou:67,verbatim:75,version:[17,24,53],view:[5,57],vm_comput:64,vo:51,vocabulari:29,vs:[43,55,57],wai:[54,55],warn:[20,53,74],weak:14,well:[27,34],what:11,when:[44,46,57],wildcard:[46,57],wlog:57,work:[11,53,66],write:[46,65,74],your:53,zifi:5}}) \ No newline at end of file +Search.setIndex({docnames:["addendum/canonical-structures","addendum/extended-pattern-matching","addendum/extraction","addendum/generalized-rewriting","addendum/implicit-coercions","addendum/micromega","addendum/miscellaneous-extensions","addendum/nsatz","addendum/parallel-proof-processing","addendum/program","addendum/rewrite-rules","addendum/ring","addendum/sprop","addendum/type-classes","addendum/universe-polymorphism","appendix/history-and-changes/index","appendix/indexes/index","changes","coq-attrindex","coq-cmdindex","coq-exnindex","coq-optindex","coq-tacindex","genindex","history","index","language/cic","language/coq-library","language/core/assumptions","language/core/basic","language/core/coinductive","language/core/conversion","language/core/definitions","language/core/index","language/core/inductive","language/core/modules","language/core/primitive","language/core/records","language/core/sections","language/core/sorts","language/core/variants","language/extensions/arguments-command","language/extensions/canonical","language/extensions/evars","language/extensions/implicit-arguments","language/extensions/index","language/extensions/match","language/gallina-extensions","language/gallina-specification-language","language/module-system","license","practical-tools/coq-commands","practical-tools/coqide","practical-tools/utilities","proof-engine/ltac","proof-engine/ltac2","proof-engine/proof-handling","proof-engine/ssreflect-proof-language","proof-engine/tactics","proof-engine/vernacular-commands","proofs/automatic-tactics/auto","proofs/automatic-tactics/index","proofs/automatic-tactics/logic","proofs/creating-tactics/index","proofs/writing-proofs/equality","proofs/writing-proofs/index","proofs/writing-proofs/proof-mode","proofs/writing-proofs/reasoning-inductives","proofs/writing-proofs/rewriting","std-glossindex","user-extensions/proof-schemes","user-extensions/syntax-extensions","using/libraries/funind","using/libraries/index","using/libraries/writing","using/tools/coqdoc","using/tools/index","zebibliography"],envversion:{"coqrst.coqdomain":2,"sphinx.domains.c":2,"sphinx.domains.changeset":1,"sphinx.domains.citation":1,"sphinx.domains.cpp":5,"sphinx.domains.index":1,"sphinx.domains.javascript":2,"sphinx.domains.math":2,"sphinx.domains.python":3,"sphinx.domains.rst":2,"sphinx.domains.std":2,"sphinx.ext.todo":2,sphinx:56},filenames:["addendum/canonical-structures.rst","addendum/extended-pattern-matching.rst","addendum/extraction.rst","addendum/generalized-rewriting.rst","addendum/implicit-coercions.rst","addendum/micromega.rst","addendum/miscellaneous-extensions.rst","addendum/nsatz.rst","addendum/parallel-proof-processing.rst","addendum/program.rst","addendum/rewrite-rules.rst","addendum/ring.rst","addendum/sprop.rst","addendum/type-classes.rst","addendum/universe-polymorphism.rst","appendix/history-and-changes/index.rst","appendix/indexes/index.rst","changes.rst","coq-attrindex.rst","coq-cmdindex.rst","coq-exnindex.rst","coq-optindex.rst","coq-tacindex.rst","genindex.rst","history.rst","index.rst","language/cic.rst","language/coq-library.rst","language/core/assumptions.rst","language/core/basic.rst","language/core/coinductive.rst","language/core/conversion.rst","language/core/definitions.rst","language/core/index.rst","language/core/inductive.rst","language/core/modules.rst","language/core/primitive.rst","language/core/records.rst","language/core/sections.rst","language/core/sorts.rst","language/core/variants.rst","language/extensions/arguments-command.rst","language/extensions/canonical.rst","language/extensions/evars.rst","language/extensions/implicit-arguments.rst","language/extensions/index.rst","language/extensions/match.rst","language/gallina-extensions.rst","language/gallina-specification-language.rst","language/module-system.rst","license.rst","practical-tools/coq-commands.rst","practical-tools/coqide.rst","practical-tools/utilities.rst","proof-engine/ltac.rst","proof-engine/ltac2.rst","proof-engine/proof-handling.rst","proof-engine/ssreflect-proof-language.rst","proof-engine/tactics.rst","proof-engine/vernacular-commands.rst","proofs/automatic-tactics/auto.rst","proofs/automatic-tactics/index.rst","proofs/automatic-tactics/logic.rst","proofs/creating-tactics/index.rst","proofs/writing-proofs/equality.rst","proofs/writing-proofs/index.rst","proofs/writing-proofs/proof-mode.rst","proofs/writing-proofs/reasoning-inductives.rst","proofs/writing-proofs/rewriting.rst","std-glossindex.rst","user-extensions/proof-schemes.rst","user-extensions/syntax-extensions.rst","using/libraries/funind.rst","using/libraries/index.rst","using/libraries/writing.rst","using/tools/coqdoc.rst","using/tools/index.rst","zebibliography.rst"],objects:{"":[[71,0,1,"coq:exn.'via'-and-'abstract'-cannot-be-used-together","'via' and 'abstract' cannot be used together"],[54,1,1,"coq:tacn.+-(backtracking-branching)","+ (backtracking branching)"],[57,1,1,"coq:tacn.=>","=>"],[66,3,1,"coq:cmd.Abort","Abort"],[59,3,1,"coq:cmd.About","About"],[71,2,1,"coq:warn.Activation-of-abbreviations-does-not-expect-mentioning-a-grammar-entry","Activation of abbreviations does not expect mentioning a grammar entry"],[71,2,1,"coq:warn.Activation-of-abbreviations-does-not-expect-mentioning-a-scope","Activation of abbreviations does not expect mentioning a scope"],[29,3,1,"coq:cmd.Add","Add"],[11,3,1,"coq:cmd.Add-Field","Add Field"],[3,3,1,"coq:cmd.Add-Morphism","Add Morphism"],[3,3,1,"coq:cmd.Add-Parametric-Morphism","Add Parametric Morphism"],[3,3,1,"coq:cmd.Add-Parametric-Relation","Add Parametric Relation"],[3,3,1,"coq:cmd.Add-Parametric-Setoid","Add Parametric Setoid"],[3,3,1,"coq:cmd.Add-Relation","Add Relation"],[11,3,1,"coq:cmd.Add-Ring","Add Ring"],[3,3,1,"coq:cmd.Add-Setoid","Add Setoid"],[5,3,1,"coq:cmd.Add-Zify","Add Zify"],[9,3,1,"coq:cmd.Admit-Obligations","Admit Obligations"],[66,3,1,"coq:cmd.Admitted","Admitted"],[12,4,1,"coq:flag.Allow-StrictProp","Allow StrictProp"],[44,0,1,"coq:exn.Argument-at-position-\u2018natural\u2019-is-mentioned-more-than-once","Argument at position \u2018natural\u2019 is mentioned more than once"],[54,0,1,"coq:exn.Argument-of-match-does-not-evaluate-to-a-term","Argument of match does not evaluate to a term"],[41,3,1,"coq:cmd.Arguments","Arguments"],[44,0,1,"coq:exn.Arguments-given-by-name-or-position-not-supported-in-explicit-mode","Arguments given by name or position not supported in explicit mode"],[11,0,1,"coq:exn.Arguments-of-ring_simplify-do-not-have-all-the-same-type","Arguments of ring_simplify do not have all the same type"],[41,0,1,"coq:exn.Arguments-of-section-variables-such-as-\u2018name\u2019-may-not-be-renamed","Arguments of section variables such as \u2018name\u2019 may not be renamed"],[46,4,1,"coq:flag.Asymmetric-Patterns","Asymmetric Patterns"],[66,0,1,"coq:exn.Attempt-to-save-an-incomplete-proof","Attempt to save an incomplete proof"],[29,3,1,"coq:cmd.Attributes","Attributes"],[34,4,1,"coq:flag.Auto-Template-Polymorphism","Auto Template Polymorphism"],[34,4,1,"coq:flag.Automatic-Proposition-Inductives","Automatic Proposition Inductives"],[34,2,1,"coq:warn.Automatically-declaring-\u2018ident\u2019-as-template-polymorphic","Automatically declaring \u2018ident\u2019 as template polymorphic"],[28,3,1,"coq:cmd.Axiom","Axiom"],[28,3,1,"coq:cmd.Axioms","Axioms"],[59,3,1,"coq:cmd.Back","Back"],[59,3,1,"coq:cmd.BackTo","BackTo"],[11,0,1,"coq:exn.Bad-lemma-for-decidability-of-equality","Bad lemma for decidability of equality"],[59,0,1,"coq:exn.Bad-magic-number","Bad magic number"],[64,0,1,"coq:exn.Bad-occurrence-number-of-\u2018qualid\u2019","Bad occurrence number of \u2018qualid\u2019"],[12,2,1,"coq:warn.Bad-relevance","Bad relevance"],[11,0,1,"coq:exn.Bad-ring-structure","Bad ring structure"],[71,3,1,"coq:cmd.Bind-Scope","Bind Scope"],[67,4,1,"coq:flag.Boolean-Equality-Schemes","Boolean Equality Schemes"],[5,5,1,"coq:thm.Bound-on-the-ceiling-function","Bound on the ceiling function"],[66,0,1,"coq:exn.Brackets-do-not-support-multi-goal-selectors","Brackets do not support multi-goal selectors"],[66,6,1,"coq:opt.Bullet-Behavior","Bullet Behavior"],[72,2,1,"coq:warn.Cannot-build-functional-inversion-principle","Cannot build functional inversion principle"],[58,0,1,"coq:exn.Cannot-change-\u2018ident\u2019,-it-is-used-in-conclusion","Cannot change \u2018ident\u2019, it is used in conclusion"],[58,0,1,"coq:exn.Cannot-change-\u2018ident\u2019,-it-is-used-in-hypothesis-\u2018ident\u2019","Cannot change \u2018ident\u2019, it is used in hypothesis \u2018ident\u2019"],[60,0,1,"coq:exn.Cannot-coerce-\u2018qualid\u2019-to-an-evaluable-reference","Cannot coerce \u2018qualid\u2019 to an evaluable reference"],[72,2,1,"coq:warn.Cannot-define-graph-for-\u2018ident\u2019","Cannot define graph for \u2018ident\u2019"],[72,2,1,"coq:warn.Cannot-define-principle(s)-for-\u2018ident\u2019","Cannot define principle(s) for \u2018ident\u2019"],[11,0,1,"coq:exn.Cannot-find-a-declared-ring-structure-for-equality-\u2018term\u2019","Cannot find a declared ring structure for equality \u2018term\u2019"],[11,0,1,"coq:exn.Cannot-find-a-declared-ring-structure-over-\u2018term\u2019","Cannot find a declared ring structure over \u2018term\u2019"],[64,0,1,"coq:exn.Cannot-find-a-relation-to-rewrite","Cannot find a relation to rewrite"],[64,0,1,"coq:exn.Cannot-find-any-non-recursive-equality-over-\u2018ident\u2019","Cannot find any non-recursive equality over \u2018ident\u2019"],[72,0,1,"coq:exn.Cannot-find-induction-information-on-\u2018qualid\u2019","Cannot find induction information on \u2018qualid\u2019"],[72,0,1,"coq:exn.Cannot-find-inversion-information-for-hypothesis-\u2018ident\u2019","Cannot find inversion information for hypothesis \u2018ident\u2019"],[59,0,1,"coq:exn.Cannot-find-library-foo-in-loadpath","Cannot find library foo in loadpath"],[4,0,1,"coq:exn.Cannot-find-the-source-class-of-\u2018qualid\u2019","Cannot find the source class of \u2018qualid\u2019"],[4,0,1,"coq:exn.Cannot-find-the-target-class","Cannot find the target class"],[35,2,1,"coq:warn.Cannot-import-local-constant,-it-will-be-ignored","Cannot import local constant, it will be ignored"],[71,0,1,"coq:exn.Cannot-interpret-in-\u2018scope_name\u2019-because-\u2018qualid\u2019-could-not-be-found-in-the-current-environment","Cannot interpret in \u2018scope_name\u2019 because \u2018qualid\u2019 could not be found in the current environment"],[71,0,1,"coq:exn.Cannot-interpret-this-number-as-a-value-of-type-\u2018type\u2019","Cannot interpret this number as a value of type \u2018type\u2019"],[71,0,1,"coq:exn.Cannot-interpret-this-string-as-a-value-of-type-\u2018type\u2019","Cannot interpret this string as a value of type \u2018type\u2019"],[59,0,1,"coq:exn.Cannot-load-\u2018qualid\u2019:-no-physical-path-bound-to-\u2018dirpath\u2019","Cannot load \u2018qualid\u2019: no physical path bound to \u2018dirpath\u2019"],[58,0,1,"coq:exn.Cannot-move-\u2018ident\u2019-after-\u2018ident\u2019:-it-depends-on-\u2018ident\u2019","Cannot move \u2018ident\u2019 after \u2018ident\u2019: it depends on \u2018ident\u2019"],[58,0,1,"coq:exn.Cannot-move-\u2018ident\u2019-after-\u2018ident\u2019:-it-occurs-in-the-type-of-\u2018ident\u2019","Cannot move \u2018ident\u2019 after \u2018ident\u2019: it occurs in the type of \u2018ident\u2019"],[62,0,1,"coq:exn.Cannot-recognize-a-boolean-equality","Cannot recognize a boolean equality"],[67,0,1,"coq:exn.Cannot-recognize-a-statement-based-on-\u2018reference\u2019","Cannot recognize a statement based on \u2018reference\u2019"],[4,0,1,"coq:exn.Cannot-recognize-\u2018coercion_class\u2019-as-a-source-class-of-\u2018qualid\u2019","Cannot recognize \u2018coercion_class\u2019 as a source class of \u2018qualid\u2019"],[64,0,1,"coq:exn.Cannot-turn-[inductive|constructor]-into-an-evaluable-reference","Cannot turn [inductive|constructor] into an evaluable reference"],[72,0,1,"coq:exn.Cannot-use-mutual-definition-with-well-founded-recursion-or-measure","Cannot use mutual definition with well-founded recursion or measure"],[42,3,1,"coq:cmd.Canonical-Structure","Canonical Structure"],[59,0,1,"coq:exn.Can\u2019t-find-file-\u2018ident\u2019-on-loadpath","Can\u2019t find file \u2018ident\u2019 on loadpath"],[67,4,1,"coq:flag.Case-Analysis-Schemes","Case Analysis Schemes"],[5,5,1,"coq:thm.Case-split","Case split"],[40,0,1,"coq:exn.Casts-are-not-supported-in-this-pattern","Casts are not supported in this pattern"],[2,3,1,"coq:cmd.Cd","Cd"],[59,3,1,"coq:cmd.Check","Check"],[13,3,1,"coq:cmd.Class","Class"],[71,3,1,"coq:cmd.Close-Scope","Close Scope"],[30,3,1,"coq:cmd.CoFixpoint","CoFixpoint"],[30,3,1,"coq:cmd.CoInductive","CoInductive"],[4,3,1,"coq:cmd.Coercion","Coercion"],[66,3,1,"coq:cmd.Collection","Collection"],[67,3,1,"coq:cmd.Combined-Scheme","Combined Scheme"],[29,3,1,"coq:cmd.Comments","Comments"],[64,3,1,"coq:cmd.Compute","Compute"],[54,0,1,"coq:exn.Condition-not-satisfied","Condition not satisfied"],[28,3,1,"coq:cmd.Conjecture","Conjecture"],[28,3,1,"coq:cmd.Conjectures","Conjectures"],[14,3,1,"coq:cmd.Constraint","Constraint"],[38,3,1,"coq:cmd.Context","Context"],[44,4,1,"coq:flag.Contextual-Implicit","Contextual Implicit"],[51,4,1,"coq:flag.Coqtop-Exit-On-Error","Coqtop Exit On Error"],[32,3,1,"coq:cmd.Corollary","Corollary"],[60,3,1,"coq:cmd.Create-HintDb","Create HintDb"],[14,7,1,"coq:attr.Cumulative","Cumulative"],[14,4,1,"coq:flag.Cumulativity-Weak-Constraints","Cumulativity Weak Constraints"],[54,3,1,"coq:cmd.Debug","Debug"],[59,6,1,"coq:opt.Debug","Debug"],[60,4,1,"coq:flag.Debug-Auto","Debug Auto"],[60,4,1,"coq:flag.Debug-Eauto","Debug Eauto"],[57,4,1,"coq:flag.Debug-SsrMatching","Debug SsrMatching"],[57,4,1,"coq:flag.Debug-Ssreflect","Debug Ssreflect"],[60,4,1,"coq:flag.Debug-Trivial","Debug Trivial"],[54,0,1,"coq:exn.Debug-mode-not-available-in-the-IDE","Debug mode not available in the IDE"],[67,4,1,"coq:flag.Decidable-Equality-Schemes","Decidable Equality Schemes"],[71,3,1,"coq:cmd.Declare-Custom-Entry","Declare Custom Entry"],[64,3,1,"coq:cmd.Declare-Equivalent-Keys","Declare Equivalent Keys"],[13,3,1,"coq:cmd.Declare-Instance","Declare Instance"],[64,3,1,"coq:cmd.Declare-Left-Step","Declare Left Step"],[59,3,1,"coq:cmd.Declare-ML-Module","Declare ML Module"],[35,3,1,"coq:cmd.Declare-Module","Declare Module"],[3,3,1,"coq:cmd.Declare-Morphism","Declare Morphism"],[64,3,1,"coq:cmd.Declare-Reduction","Declare Reduction"],[64,3,1,"coq:cmd.Declare-Right-Step","Declare Right Step"],[71,3,1,"coq:cmd.Declare-Scope","Declare Scope"],[60,2,1,"coq:warn.Declaring-arbitrary-terms-as-hints-is-fragile-and-deprecated;-it-is-recommended-to-declare-a-toplevel-constant-instead","Declaring arbitrary terms as hints is fragile and deprecated; it is recommended to declare a toplevel constant instead"],[58,6,1,"coq:opt.Default-Goal-Selector","Default Goal Selector"],[66,6,1,"coq:opt.Default-Proof-Mode","Default Proof Mode"],[66,6,1,"coq:opt.Default-Proof-Using","Default Proof Using"],[59,6,1,"coq:opt.Default-Timeout","Default Timeout"],[66,3,1,"coq:cmd.Defined","Defined"],[32,3,1,"coq:cmd.Definition","Definition"],[12,4,1,"coq:flag.Definitional-UIP","Definitional UIP"],[71,3,1,"coq:cmd.Delimit-Scope","Delimit Scope"],[34,4,1,"coq:flag.Dependent-Proposition-Eliminators","Dependent Proposition Eliminators"],[6,3,1,"coq:cmd.Derive","Derive"],[67,3,1,"coq:cmd.Derive-Dependent-Inversion","Derive Dependent Inversion"],[67,3,1,"coq:cmd.Derive-Dependent-Inversion_clear","Derive Dependent Inversion_clear"],[67,3,1,"coq:cmd.Derive-Inversion","Derive Inversion"],[67,3,1,"coq:cmd.Derive-Inversion_clear","Derive Inversion_clear"],[66,6,1,"coq:opt.Diffs","Diffs"],[71,3,1,"coq:cmd.Disable-Notation","Disable Notation"],[59,3,1,"coq:cmd.Drop","Drop"],[5,6,1,"coq:opt.Dump-Arith","Dump Arith"],[59,0,1,"coq:exn.Dynlink-error:-execution-of-module-initializers-in-the","Dynlink error: execution of module initializers in the"],[46,0,1,"coq:exn.Either-there-is-a-type-incompatibility-or-the-problem-involves-dependencies","Either there is a type incompatibility or the problem involves dependencies"],[67,4,1,"coq:flag.Elimination-Schemes","Elimination Schemes"],[71,3,1,"coq:cmd.Enable-Notation","Enable Notation"],[38,3,1,"coq:cmd.End","End"],[71,0,1,"coq:exn.End-of-quoted-string-not-followed-by-a-space-in-notation","End of quoted string not followed by a space in notation"],[64,3,1,"coq:cmd.Eval","Eval"],[32,3,1,"coq:cmd.Example","Example"],[13,3,1,"coq:cmd.Existing-Class","Existing Class"],[13,3,1,"coq:cmd.Existing-Instance","Existing Instance"],[13,3,1,"coq:cmd.Existing-Instances","Existing Instances"],[35,3,1,"coq:cmd.Export","Export"],[54,0,1,"coq:exn.Expression-does-not-evaluate-to-a-tactic","Expression does not evaluate to a tactic"],[2,3,1,"coq:cmd.Extract-Callback","Extract Callback"],[2,0,1,"coq:exn.Extract-Callback-is-supported-only-for-OCaml-extraction","Extract Callback is supported only for OCaml extraction"],[2,3,1,"coq:cmd.Extract-Constant","Extract Constant"],[2,3,1,"coq:cmd.Extract-Foreign-Constant","Extract Foreign Constant"],[2,0,1,"coq:exn.Extract-Foreign-Constant-is-supported-only-for-OCaml-extraction","Extract Foreign Constant is supported only for OCaml extraction"],[2,0,1,"coq:exn.Extract-Foreign-Constant-is-supported-only-for-functions","Extract Foreign Constant is supported only for functions"],[2,3,1,"coq:cmd.Extract-Inductive","Extract Inductive"],[2,3,1,"coq:cmd.Extract-Inlined-Constant","Extract Inlined Constant"],[2,3,1,"coq:cmd.Extraction","Extraction"],[2,4,1,"coq:flag.Extraction-AutoInline","Extraction AutoInline"],[2,3,1,"coq:cmd.Extraction-Blacklist","Extraction Blacklist"],[2,4,1,"coq:flag.Extraction-Conservative-Types","Extraction Conservative Types"],[2,6,1,"coq:opt.Extraction-File-Comment","Extraction File Comment"],[2,6,1,"coq:opt.Extraction-Flag","Extraction Flag"],[2,3,1,"coq:cmd.Extraction-Implicit","Extraction Implicit"],[2,3,1,"coq:cmd.Extraction-Inline","Extraction Inline"],[2,4,1,"coq:flag.Extraction-KeepSingleton","Extraction KeepSingleton"],[2,3,1,"coq:cmd.Extraction-Language","Extraction Language"],[2,3,1,"coq:cmd.Extraction-Library","Extraction Library"],[2,3,1,"coq:cmd.Extraction-NoInline","Extraction NoInline"],[2,4,1,"coq:flag.Extraction-Optimize","Extraction Optimize"],[2,6,1,"coq:opt.Extraction-Output-Directory","Extraction Output Directory"],[2,4,1,"coq:flag.Extraction-SafeImplicits","Extraction SafeImplicits"],[2,3,1,"coq:cmd.Extraction-TestCompile","Extraction TestCompile"],[2,4,1,"coq:flag.Extraction-TypeExpand","Extraction TypeExpand"],[32,3,1,"coq:cmd.Fact","Fact"],[59,3,1,"coq:cmd.Fail","Fail"],[54,0,1,"coq:exn.Failed-to-progress","Failed to progress"],[59,4,1,"coq:flag.Fast-Name-Printing","Fast Name Printing"],[59,0,1,"coq:exn.File-not-found-on-loadpath:-\u2018string\u2019","File not found on loadpath: \u2018string\u2019"],[59,0,1,"coq:exn.Files-processed-by-Load-cannot-leave-open-proofs","Files processed by Load cannot leave open proofs"],[9,3,1,"coq:cmd.Final-Obligation","Final Obligation"],[62,6,1,"coq:opt.Firstorder-Depth","Firstorder Depth"],[62,6,1,"coq:opt.Firstorder-Solver","Firstorder Solver"],[34,3,1,"coq:cmd.Fixpoint","Fixpoint"],[41,0,1,"coq:exn.Flag-'rename'-expected-to-rename-\u2018name\u2019-into-\u2018name\u2019","Flag 'rename' expected to rename \u2018name\u2019 into \u2018name\u2019"],[66,3,1,"coq:cmd.Focus","Focus"],[46,0,1,"coq:exn.Found-a-constructor-of-inductive-type-term-while-a-constructor-of-term-is-expected","Found a constructor of inductive type term while a constructor of term is expected"],[64,0,1,"coq:exn.Found-an-\"at\"-clause-without-\"with\"-clause","Found an "at" clause without "with" clause"],[71,2,1,"coq:warn.Found-no-matching-notation-to-enable-or-disable","Found no matching notation to enable or disable"],[64,0,1,"coq:exn.Found-no-subterm-matching-\u2018term\u2019-in-the-current-goal","Found no subterm matching \u2018term\u2019 in the current goal"],[64,0,1,"coq:exn.Found-no-subterm-matching-\u2018term\u2019-in-\u2018ident\u2019","Found no subterm matching \u2018term\u2019 in \u2018ident\u2019"],[4,0,1,"coq:exn.Found-target-class-\u2018coercion_class\u2019-instead-of-\u2018coercion_class\u2019","Found target class \u2018coercion_class\u2019 instead of \u2018coercion_class\u2019"],[59,3,1,"coq:cmd.From-\u2026-Dependency","From \u2026 Dependency"],[59,3,1,"coq:cmd.From-\u2026-Require","From \u2026 Require"],[4,0,1,"coq:exn.Funclass-cannot-be-a-source-class","Funclass cannot be a source class"],[72,3,1,"coq:cmd.Function","Function"],[72,3,1,"coq:cmd.Functional-Case","Functional Case"],[72,3,1,"coq:cmd.Functional-Scheme","Functional Scheme"],[44,3,1,"coq:cmd.Generalizable","Generalizable"],[72,3,1,"coq:cmd.Generate-graph-for","Generate graph for"],[66,3,1,"coq:cmd.Goal","Goal"],[59,4,1,"coq:flag.Guard-Checking","Guard Checking"],[66,3,1,"coq:cmd.Guarded","Guarded"],[60,3,1,"coq:cmd.Hint-Constants","Hint Constants"],[60,3,1,"coq:cmd.Hint-Constructors","Hint Constructors"],[60,3,1,"coq:cmd.Hint-Cut","Hint Cut"],[60,3,1,"coq:cmd.Hint-Extern","Hint Extern"],[60,3,1,"coq:cmd.Hint-Immediate","Hint Immediate"],[60,3,1,"coq:cmd.Hint-Mode","Hint Mode"],[60,3,1,"coq:cmd.Hint-Opaque","Hint Opaque"],[60,3,1,"coq:cmd.Hint-Projections","Hint Projections"],[60,3,1,"coq:cmd.Hint-Resolve","Hint Resolve"],[60,3,1,"coq:cmd.Hint-Rewrite","Hint Rewrite"],[60,3,1,"coq:cmd.Hint-Transparent","Hint Transparent"],[60,3,1,"coq:cmd.Hint-Unfold","Hint Unfold"],[60,3,1,"coq:cmd.Hint-Variables","Hint Variables"],[57,3,1,"coq:cmd.Hint-View-for","Hint View for"],[57,3,1,"coq:cmd.Hint-View-for-apply","Hint View for apply"],[57,3,1,"coq:cmd.Hint-View-for-move","Hint View for move"],[28,3,1,"coq:cmd.Hypotheses","Hypotheses"],[28,3,1,"coq:cmd.Hypothesis","Hypothesis"],[72,0,1,"coq:exn.Hypothesis-\u2018ident\u2019-must-contain-at-least-one-Function","Hypothesis \u2018ident\u2019 must contain at least one Function"],[66,6,1,"coq:opt.Hyps-Limit","Hyps Limit"],[62,0,1,"coq:exn.I-don\u2019t-know-how-to-handle-dependent-equality","I don\u2019t know how to handle dependent equality"],[4,3,1,"coq:cmd.Identity-Coercion","Identity Coercion"],[13,2,1,"coq:warn.Ignored-instance-declaration-for-\u201c\u2018ident\u2019\u201d:-\u201c\u2018term\u2019\u201d-is-not-a-class","Ignored instance declaration for \u201c\u2018ident\u2019\u201d: \u201c\u2018term\u2019\u201d is not a class"],[44,2,1,"coq:warn.Ignoring-implicit-binder-declaration-in-unexpected-position","Ignoring implicit binder declaration in unexpected position"],[9,0,1,"coq:exn.Ill-formed-recursive-definition","Ill-formed recursive definition"],[34,0,1,"coq:exn.Ill-formed-template-inductive-declaration:-not-polymorphic-on-any-universe","Ill-formed template inductive declaration: not polymorphic on any universe"],[44,4,1,"coq:flag.Implicit-Arguments","Implicit Arguments"],[44,3,1,"coq:cmd.Implicit-Type","Implicit Type"],[44,3,1,"coq:cmd.Implicit-Types","Implicit Types"],[35,3,1,"coq:cmd.Import","Import"],[35,3,1,"coq:cmd.Include","Include"],[35,3,1,"coq:cmd.Include-Type","Include Type"],[57,0,1,"coq:exn.Incorrect-number-of-tactics-(expected-N-tactics,-was-given-M)","Incorrect number of tactics (expected N tactics, was given M)"],[34,3,1,"coq:cmd.Inductive","Inductive"],[71,3,1,"coq:cmd.Infix","Infix"],[54,3,1,"coq:cmd.Info","Info"],[60,4,1,"coq:flag.Info-Auto","Info Auto"],[60,4,1,"coq:flag.Info-Eauto","Info Eauto"],[54,6,1,"coq:opt.Info-Level","Info Level"],[5,4,1,"coq:flag.Info-Micromega","Info Micromega"],[60,4,1,"coq:flag.Info-Trivial","Info Trivial"],[59,3,1,"coq:cmd.Inspect","Inspect"],[13,3,1,"coq:cmd.Instance","Instance"],[59,3,1,"coq:cmd.Instructions","Instructions"],[62,4,1,"coq:flag.Intuition-Negation-Unfolding","Intuition Negation Unfolding"],[59,0,1,"coq:exn.Invalid-backtrack","Invalid backtrack"],[67,8,1,"coq:table.Keep-Equalities","Keep Equalities"],[67,4,1,"coq:flag.Keep-Proof-Equalities","Keep Proof Equalities"],[64,4,1,"coq:flag.Kernel-Term-Sharing","Kernel Term Sharing"],[64,4,1,"coq:flag.Keyed-Unification","Keyed Unification"],[38,0,1,"coq:exn.Last-block-to-end-has-name-\u2018ident\u2019","Last block to end has name \u2018ident\u2019"],[32,3,1,"coq:cmd.Lemma","Lemma"],[38,3,1,"coq:cmd.Let","Let"],[38,3,1,"coq:cmd.Let-CoFixpoint","Let CoFixpoint"],[38,3,1,"coq:cmd.Let-Fixpoint","Let Fixpoint"],[5,4,1,"coq:flag.Lia-Cache","Lia Cache"],[59,3,1,"coq:cmd.Load","Load"],[59,0,1,"coq:exn.Load-is-not-supported-inside-proofs","Load is not supported inside proofs"],[59,3,1,"coq:cmd.Locate","Locate"],[59,3,1,"coq:cmd.Locate-File","Locate File"],[59,3,1,"coq:cmd.Locate-Library","Locate Library"],[59,3,1,"coq:cmd.Locate-Ltac","Locate Ltac"],[59,3,1,"coq:cmd.Locate-Ltac2","Locate Ltac2"],[59,3,1,"coq:cmd.Locate-Module","Locate Module"],[59,3,1,"coq:cmd.Locate-Term","Locate Term"],[60,6,1,"coq:opt.Loose-Hint-Behavior","Loose Hint Behavior"],[54,3,1,"coq:cmd.Ltac","Ltac"],[54,4,1,"coq:flag.Ltac-Backtrace","Ltac Backtrace"],[54,4,1,"coq:flag.Ltac-Batch-Debug","Ltac Batch Debug"],[54,4,1,"coq:flag.Ltac-Debug","Ltac Debug"],[54,4,1,"coq:flag.Ltac-Profiling","Ltac Profiling"],[55,3,1,"coq:cmd.Ltac2","Ltac2"],[55,4,1,"coq:flag.Ltac2-Backtrace","Ltac2 Backtrace"],[55,3,1,"coq:cmd.Ltac2-Check","Ltac2 Check"],[55,3,1,"coq:cmd.Ltac2-Eval","Ltac2 Eval"],[55,3,1,"coq:cmd.Ltac2-Globalize","Ltac2 Globalize"],[55,4,1,"coq:flag.Ltac2-In-Ltac1-Profiling","Ltac2 In Ltac1 Profiling"],[55,3,1,"coq:cmd.Ltac2-Notation","Ltac2 Notation"],[55,3,1,"coq:cmd.Ltac2-Notation-(abbreviation)","Ltac2 Notation (abbreviation)"],[55,3,1,"coq:cmd.Ltac2-Set","Ltac2 Set"],[55,3,1,"coq:cmd.Ltac2-Type","Ltac2 Type"],[55,4,1,"coq:flag.Ltac2-Typed-Notations","Ltac2 Typed Notations"],[55,3,1,"coq:cmd.Ltac2-external","Ltac2 external"],[44,2,1,"coq:warn.Making-shadowed-name-of-implicit-argument-accessible-by-position","Making shadowed name of implicit argument accessible by position"],[66,4,1,"coq:flag.Mangle-Names","Mangle Names"],[66,4,1,"coq:flag.Mangle-Names-Light","Mangle Names Light"],[66,6,1,"coq:opt.Mangle-Names-Prefix","Mangle Names Prefix"],[44,4,1,"coq:flag.Maximal-Implicit-Insertion","Maximal Implicit Insertion"],[71,0,1,"coq:exn.Missing-mapping-for-constructor-\u2018qualid\u2019","Missing mapping for constructor \u2018qualid\u2019"],[35,3,1,"coq:cmd.Module","Module"],[35,3,1,"coq:cmd.Module-Type","Module Type"],[59,0,1,"coq:exn.Module/section-\u2018qualid\u2019-not-found","Module/section \u2018qualid\u2019 not found"],[14,7,1,"coq:attr.Monomorphic","Monomorphic"],[71,0,1,"coq:exn.More-than-one-interpretation-bound-to-this-notation,-confirm-with-the-\"all\"-modifier","More than one interpretation bound to this notation, confirm with the "all" modifier"],[71,0,1,"coq:exn.Multiple-'via'-options","Multiple 'via' options"],[71,0,1,"coq:exn.Multiple-'warning-after'-or-'abstract-after'-options","Multiple 'warning after' or 'abstract after' options"],[64,6,1,"coq:opt.NativeCompute-Profile-Filename","NativeCompute Profile Filename"],[64,4,1,"coq:flag.NativeCompute-Profiling","NativeCompute Profiling"],[64,4,1,"coq:flag.NativeCompute-Timing","NativeCompute Timing"],[66,4,1,"coq:flag.Nested-Proofs-Allowed","Nested Proofs Allowed"],[66,2,1,"coq:warn.New-Collection-definition-of-\u2018ident\u2019-shadows-the-previous-one","New Collection definition of \u2018ident\u2019 shadows the previous one"],[9,3,1,"coq:cmd.Next-Obligation","Next Obligation"],[5,4,1,"coq:flag.Nia-Cache","Nia Cache"],[54,0,1,"coq:exn.No-applicable-tactic","No applicable tactic"],[72,0,1,"coq:exn.No-argument-name-\u2018ident\u2019","No argument name \u2018ident\u2019"],[54,0,1,"coq:exn.No-evars","No evars"],[35,0,1,"coq:exn.No-field-named-\u2018ident\u2019-in-\u2018qualid\u2019","No field named \u2018ident\u2019 in \u2018qualid\u2019"],[66,0,1,"coq:exn.No-focused-proof","No focused proof"],[66,0,1,"coq:exn.No-focused-proof-(No-proof-editing-in-progress)","No focused proof (No proof-editing in progress)"],[66,0,1,"coq:exn.No-focused-proof-to-restart","No focused proof to restart"],[64,0,1,"coq:exn.No-head-constant-to-reduce","No head constant to reduce"],[54,0,1,"coq:exn.No-matching-clauses-for-match","No matching clauses for match"],[54,0,1,"coq:exn.No-matching-clauses-for-match-goal","No matching clauses for match goal"],[71,0,1,"coq:exn.No-notation-provided","No notation provided"],[67,0,1,"coq:exn.No-primitive-equality-found","No primitive equality found"],[58,0,1,"coq:exn.No-product-even-after-head-reduction","No product even after head-reduction"],[3,0,1,"coq:exn.No-progress-made","No progress made"],[58,0,1,"coq:exn.No-quantified-hypothesis-named-\u2018ident\u2019-in-current-goal-even-after-head-reduction","No quantified hypothesis named \u2018ident\u2019 in current goal even after head-reduction"],[58,0,1,"coq:exn.No-such-assumption","No such assumption"],[58,0,1,"coq:exn.No-such-binder","No such binder"],[58,0,1,"coq:exn.No-such-bound-variable-\u2018ident\u2019-(no-bound-variables-at-all-in-the-expression)","No such bound variable \u2018ident\u2019 (no bound variables at all in the expression)"],[66,0,1,"coq:exn.No-such-goal","No such goal"],[66,0,1,"coq:exn.No-such-goal-(\u2018ident\u2019)","No such goal (\u2018ident\u2019)"],[66,0,1,"coq:exn.No-such-goal-(\u2018natural\u2019)","No such goal (\u2018natural\u2019)"],[58,0,1,"coq:exn.No-such-hypothesis:-\u2018ident\u2019","No such hypothesis: \u2018ident\u2019"],[58,0,1,"coq:exn.No-\u2018natural\u2019-th-non-dependent-hypothesis-in-current-goal-even-after-head-reduction","No \u2018natural\u2019-th non dependent hypothesis in current goal even after head-reduction"],[46,0,1,"coq:exn.Non-exhaustive-pattern-matching","Non exhaustive pattern matching"],[9,0,1,"coq:exn.Non-extensible-universe-declaration-not-supported-with-monomorphic-Program-Definition","Non extensible universe declaration not supported with monomorphic Program Definition"],[34,0,1,"coq:exn.Non-strictly-positive-occurrence-of-\u2018ident\u2019-in-\u2018type\u2019","Non strictly positive occurrence of \u2018ident\u2019 in \u2018type\u2019"],[14,7,1,"coq:attr.NonCumulative","NonCumulative"],[67,4,1,"coq:flag.Nonrecursive-Elimination-Schemes","Nonrecursive Elimination Schemes"],[54,0,1,"coq:exn.Not-a-context-variable","Not a context variable"],[67,0,1,"coq:exn.Not-a-discriminable-equality","Not a discriminable equality"],[67,0,1,"coq:exn.Not-a-negated-primitive-equality","Not a negated primitive equality"],[11,0,1,"coq:exn.Not-a-valid-ring-equation","Not a valid ring equation"],[54,0,1,"coq:exn.Not-a-variable-or-hypothesis","Not a variable or hypothesis"],[54,0,1,"coq:exn.Not-an-evar","Not an evar"],[58,0,1,"coq:exn.Not-an-exact-proof","Not an exact proof"],[67,0,1,"coq:exn.Not-an-inductive-goal-with-1-constructor","Not an inductive goal with 1 constructor"],[67,0,1,"coq:exn.Not-an-inductive-goal-with-2-constructors","Not an inductive goal with 2 constructors"],[67,0,1,"coq:exn.Not-an-inductive-product","Not an inductive product"],[64,0,1,"coq:exn.Not-convertible","Not convertible"],[67,0,1,"coq:exn.Not-enough-constructors","Not enough constructors"],[44,0,1,"coq:exn.Not-enough-non-implicit-arguments-to-accept-the-argument-bound-to-\u2018ident\u2019","Not enough non implicit arguments to accept the argument bound to \u2018ident\u2019"],[44,0,1,"coq:exn.Not-enough-non-implicit-arguments-to-accept-the-argument-bound-to-\u2018natural\u2019","Not enough non implicit arguments to accept the argument bound to \u2018natural\u2019"],[54,0,1,"coq:exn.Not-equal","Not equal"],[54,0,1,"coq:exn.Not-equal-(due-to-universes)","Not equal (due to universes)"],[54,0,1,"coq:exn.Not-ground","Not ground"],[72,0,1,"coq:exn.Not-the-right-number-of-induction-arguments","Not the right number of induction arguments"],[58,0,1,"coq:exn.Not-the-right-number-of-missing-arguments-(expected-\u2018natural\u2019)","Not the right number of missing arguments (expected \u2018natural\u2019)"],[71,3,1,"coq:cmd.Notation","Notation"],[71,3,1,"coq:cmd.Notation-(abbreviation)","Notation (abbreviation)"],[55,0,1,"coq:exn.Notation-levels-must-range-between-0-and-6","Notation levels must range between 0 and 6"],[67,0,1,"coq:exn.Nothing-to-inject","Nothing to inject"],[3,0,1,"coq:exn.Nothing-to-rewrite","Nothing to rewrite"],[5,4,1,"coq:flag.Nra-Cache","Nra Cache"],[71,3,1,"coq:cmd.Number-Notation","Number Notation"],[9,3,1,"coq:cmd.Obligation","Obligation"],[9,3,1,"coq:cmd.Obligation-Tactic","Obligation Tactic"],[9,3,1,"coq:cmd.Obligations","Obligations"],[64,3,1,"coq:cmd.Opaque","Opaque"],[71,3,1,"coq:cmd.Open-Scope","Open Scope"],[66,3,1,"coq:cmd.Optimize-Heap","Optimize Heap"],[66,3,1,"coq:cmd.Optimize-Proof","Optimize Proof"],[28,3,1,"coq:cmd.Parameter","Parameter"],[28,3,1,"coq:cmd.Parameters","Parameters"],[44,4,1,"coq:flag.Parsing-Explicit","Parsing Explicit"],[14,7,1,"coq:attr.Polymorphic","Polymorphic"],[14,4,1,"coq:flag.Polymorphic-Inductive-Cumulativity","Polymorphic Inductive Cumulativity"],[14,0,1,"coq:exn.Polymorphic-universe-constraints-can-only-be-declared-inside-sections,-use-Monomorphic-Constraint-instead","Polymorphic universe constraints can only be declared inside sections, use Monomorphic Constraint instead"],[14,0,1,"coq:exn.Polymorphic-universes-can-only-be-declared-inside-sections,-use-Monomorphic-Universe-instead","Polymorphic universes can only be declared inside sections, use Monomorphic Universe instead"],[59,4,1,"coq:flag.Positivity-Checking","Positivity Checking"],[57,3,1,"coq:cmd.Prenex-Implicits","Prenex Implicits"],[9,3,1,"coq:cmd.Preterm","Preterm"],[59,3,1,"coq:cmd.Primitive","Primitive"],[37,4,1,"coq:flag.Primitive-Projections","Primitive Projections"],[59,3,1,"coq:cmd.Print","Print"],[59,3,1,"coq:cmd.Print-All","Print All"],[59,3,1,"coq:cmd.Print-All-Dependencies","Print All Dependencies"],[59,3,1,"coq:cmd.Print-Assumptions","Print Assumptions"],[42,3,1,"coq:cmd.Print-Canonical-Projections","Print Canonical Projections"],[4,3,1,"coq:cmd.Print-Classes","Print Classes"],[4,3,1,"coq:cmd.Print-Coercion-Paths","Print Coercion Paths"],[4,3,1,"coq:cmd.Print-Coercions","Print Coercions"],[71,3,1,"coq:cmd.Print-Custom-Grammar","Print Custom Grammar"],[66,3,1,"coq:cmd.Print-Debug-GC","Print Debug GC"],[64,3,1,"coq:cmd.Print-Equivalent-Keys","Print Equivalent Keys"],[2,3,1,"coq:cmd.Print-Extraction-Blacklist","Print Extraction Blacklist"],[2,3,1,"coq:cmd.Print-Extraction-Callback","Print Extraction Callback"],[2,3,1,"coq:cmd.Print-Extraction-Foreign","Print Extraction Foreign"],[2,3,1,"coq:cmd.Print-Extraction-Inline","Print Extraction Inline"],[11,3,1,"coq:cmd.Print-Fields","Print Fields"],[62,3,1,"coq:cmd.Print-Firstorder-Solver","Print Firstorder Solver"],[71,3,1,"coq:cmd.Print-Grammar","Print Grammar"],[4,3,1,"coq:cmd.Print-Graph","Print Graph"],[60,3,1,"coq:cmd.Print-Hint","Print Hint"],[60,3,1,"coq:cmd.Print-HintDb","Print HintDb"],[44,3,1,"coq:cmd.Print-Implicit","Print Implicit"],[13,3,1,"coq:cmd.Print-Instances","Print Instances"],[71,3,1,"coq:cmd.Print-Keywords","Print Keywords"],[59,3,1,"coq:cmd.Print-Libraries","Print Libraries"],[59,3,1,"coq:cmd.Print-LoadPath","Print LoadPath"],[54,3,1,"coq:cmd.Print-Ltac","Print Ltac"],[54,3,1,"coq:cmd.Print-Ltac-Signatures","Print Ltac Signatures"],[55,3,1,"coq:cmd.Print-Ltac2","Print Ltac2"],[55,3,1,"coq:cmd.Print-Ltac2-Signatures","Print Ltac2 Signatures"],[55,3,1,"coq:cmd.Print-Ltac2-Type","Print Ltac2 Type"],[59,3,1,"coq:cmd.Print-ML-Modules","Print ML Modules"],[59,3,1,"coq:cmd.Print-ML-Path","Print ML Path"],[35,3,1,"coq:cmd.Print-Module","Print Module"],[35,3,1,"coq:cmd.Print-Module-Type","Print Module Type"],[35,3,1,"coq:cmd.Print-Namespace","Print Namespace"],[71,3,1,"coq:cmd.Print-Notation","Print Notation"],[59,3,1,"coq:cmd.Print-Opaque-Dependencies","Print Opaque Dependencies"],[29,3,1,"coq:cmd.Print-Options","Print Options"],[59,3,1,"coq:cmd.Print-Registered","Print Registered"],[59,3,1,"coq:cmd.Print-Registered-Schemes","Print Registered Schemes"],[60,3,1,"coq:cmd.Print-Rewrite-HintDb","Print Rewrite HintDb"],[11,3,1,"coq:cmd.Print-Rings","Print Rings"],[71,3,1,"coq:cmd.Print-Scope","Print Scope"],[71,3,1,"coq:cmd.Print-Scopes","Print Scopes"],[59,3,1,"coq:cmd.Print-Section","Print Section"],[64,3,1,"coq:cmd.Print-Strategies","Print Strategies"],[64,3,1,"coq:cmd.Print-Strategy","Print Strategy"],[29,3,1,"coq:cmd.Print-Table","Print Table"],[29,3,1,"coq:cmd.Print-Tables","Print Tables"],[59,3,1,"coq:cmd.Print-Transparent-Dependencies","Print Transparent Dependencies"],[13,3,1,"coq:cmd.Print-Typeclasses","Print Typeclasses"],[59,3,1,"coq:cmd.Print-Typing-Flags","Print Typing Flags"],[14,3,1,"coq:cmd.Print-Universes","Print Universes"],[71,3,1,"coq:cmd.Print-Visibility","Print Visibility"],[59,4,1,"coq:flag.Printing-All","Printing All"],[46,4,1,"coq:flag.Printing-Allow-Match-Default-Clause","Printing Allow Match Default Clause"],[4,8,1,"coq:table.Printing-Coercion","Printing Coercion"],[4,4,1,"coq:flag.Printing-Coercions","Printing Coercions"],[59,4,1,"coq:flag.Printing-Compact-Contexts","Printing Compact Contexts"],[37,8,1,"coq:table.Printing-Constructor","Printing Constructor"],[59,4,1,"coq:flag.Printing-Dependent-Evars-Line","Printing Dependent Evars Line"],[59,6,1,"coq:opt.Printing-Depth","Printing Depth"],[43,4,1,"coq:flag.Printing-Existential-Instances","Printing Existential Instances"],[46,4,1,"coq:flag.Printing-Factorizable-Match-Patterns","Printing Factorizable Match Patterns"],[27,4,1,"coq:flag.Printing-Float","Printing Float"],[66,4,1,"coq:flag.Printing-Goal-Names","Printing Goal Names"],[66,4,1,"coq:flag.Printing-Goal-Tags","Printing Goal Tags"],[46,8,1,"coq:table.Printing-If","Printing If"],[44,4,1,"coq:flag.Printing-Implicit","Printing Implicit"],[44,4,1,"coq:flag.Printing-Implicit-Defensive","Printing Implicit Defensive"],[46,8,1,"coq:table.Printing-Let","Printing Let"],[46,4,1,"coq:flag.Printing-Match-All-Subterms","Printing Match All Subterms"],[46,4,1,"coq:flag.Printing-Matching","Printing Matching"],[71,4,1,"coq:flag.Printing-Notations","Printing Notations"],[71,4,1,"coq:flag.Printing-Parentheses","Printing Parentheses"],[37,4,1,"coq:flag.Printing-Primitive-Projection-Parameters","Printing Primitive Projection Parameters"],[37,4,1,"coq:flag.Printing-Projections","Printing Projections"],[71,4,1,"coq:flag.Printing-Raw-Literals","Printing Raw Literals"],[37,8,1,"coq:table.Printing-Record","Printing Record"],[37,4,1,"coq:flag.Printing-Records","Printing Records"],[12,4,1,"coq:flag.Printing-Relevance-Marks","Printing Relevance Marks"],[46,4,1,"coq:flag.Printing-Synth","Printing Synth"],[59,4,1,"coq:flag.Printing-Unfocused","Printing Unfocused"],[37,4,1,"coq:flag.Printing-Unfolded-Projection-As-Match","Printing Unfolded Projection As Match"],[14,4,1,"coq:flag.Printing-Universes","Printing Universes"],[44,4,1,"coq:flag.Printing-Use-Implicit-Types","Printing Use Implicit Types"],[59,6,1,"coq:opt.Printing-Width","Printing Width"],[46,4,1,"coq:flag.Printing-Wildcard","Printing Wildcard"],[40,7,1,"coq:attr.Private","Private"],[14,4,1,"coq:flag.Private-Polymorphic-Universes","Private Polymorphic Universes"],[59,3,1,"coq:cmd.Profile","Profile"],[9,7,1,"coq:attr.Program","Program"],[9,4,1,"coq:flag.Program-Cases","Program Cases"],[9,4,1,"coq:flag.Program-Generalized-Coercion","Program Generalized Coercion"],[9,4,1,"coq:flag.Program-Mode","Program Mode"],[66,3,1,"coq:cmd.Proof","Proof"],[66,3,1,"coq:cmd.Proof-Mode","Proof Mode"],[66,3,1,"coq:cmd.Proof-`term`","Proof `term`"],[66,3,1,"coq:cmd.Proof-using","Proof using"],[60,3,1,"coq:cmd.Proof-with","Proof with"],[32,3,1,"coq:cmd.Property","Property"],[32,3,1,"coq:cmd.Proposition","Proposition"],[5,5,1,"coq:thm.Psatz","Psatz"],[2,3,1,"coq:cmd.Pwd","Pwd"],[66,3,1,"coq:cmd.Qed","Qed"],[59,3,1,"coq:cmd.Quit","Quit"],[37,3,1,"coq:cmd.Record","Record"],[37,0,1,"coq:exn.Records-declared-with-the-keyword-Record-or-Structure-cannot-be-recursive","Records declared with the keyword Record or Structure cannot be recursive"],[2,3,1,"coq:cmd.Recursive-Extraction","Recursive Extraction"],[2,3,1,"coq:cmd.Recursive-Extraction-Library","Recursive Extraction Library"],[59,3,1,"coq:cmd.Redirect","Redirect"],[59,3,1,"coq:cmd.Register","Register"],[59,3,1,"coq:cmd.Register-Inline","Register Inline"],[59,3,1,"coq:cmd.Register-Scheme","Register Scheme"],[64,4,1,"coq:flag.Regular-Subst-Tactic","Regular Subst Tactic"],[32,3,1,"coq:cmd.Remark","Remark"],[29,3,1,"coq:cmd.Remove","Remove"],[60,3,1,"coq:cmd.Remove-Hints","Remove Hints"],[59,3,1,"coq:cmd.Require","Require"],[59,3,1,"coq:cmd.Require-Export","Require Export"],[59,3,1,"coq:cmd.Require-Import","Require Import"],[71,3,1,"coq:cmd.Reserved-Infix","Reserved Infix"],[71,3,1,"coq:cmd.Reserved-Notation","Reserved Notation"],[59,3,1,"coq:cmd.Reset","Reset"],[2,3,1,"coq:cmd.Reset-Extraction-Blacklist","Reset Extraction Blacklist"],[2,3,1,"coq:cmd.Reset-Extraction-Callback","Reset Extraction Callback"],[2,3,1,"coq:cmd.Reset-Extraction-Inline","Reset Extraction Inline"],[59,3,1,"coq:cmd.Reset-Initial","Reset Initial"],[54,3,1,"coq:cmd.Reset-Ltac-Profile","Reset Ltac Profile"],[66,3,1,"coq:cmd.Restart","Restart"],[44,4,1,"coq:flag.Reversible-Pattern-Implicit","Reversible Pattern Implicit"],[10,3,1,"coq:cmd.Rewrite-Rule","Rewrite Rule"],[10,3,1,"coq:cmd.Rewrite-Rules","Rewrite Rules"],[10,0,1,"coq:exn.Rewrite-rule-declaration-requires-passing-the-flag-\"-allow-rewrite-rules\"","Rewrite rule declaration requires passing the flag "-allow-rewrite-rules""],[67,4,1,"coq:flag.Rewriting-Schemes","Rewriting Schemes"],[11,0,1,"coq:exn.Ring-operation-should-be-declared-as-a-morphism","Ring operation should be declared as a morphism"],[12,0,1,"coq:exn.SProp-is-disallowed-because-the-\"Allow-StrictProp\"-flag-is-off","SProp is disallowed because the "Allow StrictProp" flag is off"],[66,3,1,"coq:cmd.Save","Save"],[67,3,1,"coq:cmd.Scheme","Scheme"],[67,3,1,"coq:cmd.Scheme-Boolean-Equality","Scheme Boolean Equality"],[67,3,1,"coq:cmd.Scheme-Equality","Scheme Equality"],[71,0,1,"coq:exn.Scope-delimiters-should-not-start-with-an-underscore","Scope delimiters should not start with an underscore"],[71,0,1,"coq:exn.Scope-names-should-not-start-with-an-underscore","Scope names should not start with an underscore"],[59,3,1,"coq:cmd.Search","Search"],[59,8,1,"coq:table.Search-Blacklist","Search Blacklist"],[59,4,1,"coq:flag.Search-Output-Name-Only","Search Output Name Only"],[59,3,1,"coq:cmd.SearchPattern","SearchPattern"],[59,3,1,"coq:cmd.SearchRewrite","SearchRewrite"],[38,3,1,"coq:cmd.Section","Section"],[64,0,1,"coq:exn.Section-variable-\u2018ident\u2019-occurs-implicitly-in-global-declaration-\u2018qualid\u2019-present-in-hypothesis-\u2018ident\u2019","Section variable \u2018ident\u2019 occurs implicitly in global declaration \u2018qualid\u2019 present in hypothesis \u2018ident\u2019"],[64,0,1,"coq:exn.Section-variable-\u2018ident\u2019-occurs-implicitly-in-global-declaration-\u2018qualid\u2019-present-in-the-conclusion","Section variable \u2018ident\u2019 occurs implicitly in global declaration \u2018qualid\u2019 present in the conclusion"],[2,3,1,"coq:cmd.Separate-Extraction","Separate Extraction"],[29,3,1,"coq:cmd.Set","Set"],[35,4,1,"coq:flag.Short-Module-Printing","Short Module Printing"],[66,3,1,"coq:cmd.Show","Show"],[66,3,1,"coq:cmd.Show-Conjectures","Show Conjectures"],[66,3,1,"coq:cmd.Show-Existentials","Show Existentials"],[2,3,1,"coq:cmd.Show-Extraction","Show Extraction"],[66,3,1,"coq:cmd.Show-Goal","Show Goal"],[66,3,1,"coq:cmd.Show-Intro","Show Intro"],[66,3,1,"coq:cmd.Show-Intros","Show Intros"],[5,3,1,"coq:cmd.Show-Lia-Profile","Show Lia Profile"],[54,3,1,"coq:cmd.Show-Ltac-Profile","Show Ltac Profile"],[66,3,1,"coq:cmd.Show-Match","Show Match"],[9,3,1,"coq:cmd.Show-Obligation-Tactic","Show Obligation Tactic"],[66,3,1,"coq:cmd.Show-Proof","Show Proof"],[66,3,1,"coq:cmd.Show-Universes","Show Universes"],[5,3,1,"coq:cmd.Show-Zify","Show Zify"],[35,0,1,"coq:exn.Signature-components-for-field-\u2018ident\u2019-do-not-match","Signature components for field \u2018ident\u2019 do not match"],[59,4,1,"coq:flag.Silent","Silent"],[9,3,1,"coq:cmd.Solve-All-Obligations","Solve All Obligations"],[9,3,1,"coq:cmd.Solve-Obligations","Solve Obligations"],[66,4,1,"coq:flag.Solve-Unification-Constraints","Solve Unification Constraints"],[57,4,1,"coq:flag.SsrHave-NoTCResolution","SsrHave NoTCResolution"],[57,4,1,"coq:flag.SsrIdents","SsrIdents"],[57,4,1,"coq:flag.SsrOldRewriteGoalsOrder","SsrOldRewriteGoalsOrder"],[57,4,1,"coq:flag.SsrRewrite","SsrRewrite"],[71,2,1,"coq:warn.Stack-overflow-or-segmentation-fault-happens-when-working-with-large-numbers-in-\u2018type\u2019-(threshold-may-vary-depending-on-your-system-limits-and-on-the-command-executed)","Stack overflow or segmentation fault happens when working with large numbers in \u2018type\u2019 (threshold may vary depending on your system limits and on the command executed)"],[64,3,1,"coq:cmd.Strategy","Strategy"],[44,4,1,"coq:flag.Strict-Implicit","Strict Implicit"],[14,4,1,"coq:flag.Strict-Universe-Declaration","Strict Universe Declaration"],[71,3,1,"coq:cmd.String-Notation","String Notation"],[44,4,1,"coq:flag.Strongly-Strict-Implicit","Strongly Strict Implicit"],[67,4,1,"coq:flag.Structural-Injection","Structural Injection"],[37,3,1,"coq:cmd.Structure","Structure"],[4,3,1,"coq:cmd.SubClass","SubClass"],[59,3,1,"coq:cmd.Succeed","Succeed"],[66,4,1,"coq:flag.Suggest-Proof-Using","Suggest Proof Using"],[10,3,1,"coq:cmd.Symbol","Symbol"],[10,3,1,"coq:cmd.Symbols","Symbols"],[71,0,1,"coq:exn.Syntax-error:-[prim:reference]-expected-after-'Notation'-(in-[vernac:command])","Syntax error: [prim:reference] expected after 'Notation' (in [vernac:command])"],[71,0,1,"coq:exn.Syntax-error:-[prim:reference]-expected-after-[prim:reference]-(in-[vernac:command])","Syntax error: [prim:reference] expected after [prim:reference] (in [vernac:command])"],[71,3,1,"coq:cmd.Tactic-Notation","Tactic Notation"],[54,0,1,"coq:exn.Tactic-failure","Tactic failure"],[54,0,1,"coq:exn.Tactic-failure-(level-\u2018natural\u2019)","Tactic failure (level \u2018natural\u2019)"],[54,0,1,"coq:exn.Tactic-failure:--succeeds","Tactic failure: <tactic closure> succeeds"],[64,0,1,"coq:exn.Tactic-failure:-Setoid-library-not-loaded","Tactic failure: Setoid library not loaded"],[64,0,1,"coq:exn.Tactic-generated-a-subgoal-identical-to-the-original-goal","Tactic generated a subgoal identical to the original goal"],[64,0,1,"coq:exn.Terms-do-not-have-convertible-types","Terms do not have convertible types"],[29,3,1,"coq:cmd.Test","Test"],[60,0,1,"coq:exn.The-\"at\"-syntax-isn't-available-yet-for-the-autorewrite-tactic","The "at" syntax isn't available yet for the autorewrite tactic"],[41,0,1,"coq:exn.The-&-modifier-may-only-occur-once","The & modifier may only occur once"],[71,2,1,"coq:warn.The-'abstract-after'-directive-has-no-effect-when-the-parsing-function-(\u2018qualid\u2019)-targets-an-option-type","The 'abstract after' directive has no effect when the parsing function (\u2018qualid\u2019) targets an option type"],[41,0,1,"coq:exn.The-'clear-implicits'-flag-must-be-omitted-if-implicit-annotations-are-given","The 'clear implicits' flag must be omitted if implicit annotations are given"],[41,0,1,"coq:exn.The-'default-implicits'-flag-is-incompatible-with-implicit-annotations","The 'default implicits' flag is incompatible with implicit annotations"],[41,0,1,"coq:exn.The-/-modifier-may-only-occur-once","The / modifier may only occur once"],[59,0,1,"coq:exn.The-command-has-not-failed!","The command has not failed!"],[34,0,1,"coq:exn.The-conclusion-of-\u2018type\u2019-is-not-valid;-it-must-be-built-from-\u2018ident\u2019","The conclusion of \u2018type\u2019 is not valid; it must be built from \u2018ident\u2019"],[46,0,1,"coq:exn.The-constructor-\u2018ident\u2019-expects-\u2018natural\u2019-arguments","The constructor \u2018ident\u2019 expects \u2018natural\u2019 arguments"],[14,0,1,"coq:exn.The-cumulative-attribute-can-only-be-used-in-a-polymorphic-context","The cumulative attribute can only be used in a polymorphic context"],[46,0,1,"coq:exn.The-elimination-predicate-term-should-be-of-arity-\u2018natural\u2019-(for-non-dependent-case)-or-\u2018natural\u2019-(for-dependent-case)","The elimination predicate term should be of arity \u2018natural\u2019 (for non dependent case) or \u2018natural\u2019 (for dependent case)"],[35,0,1,"coq:exn.The-field-\u2018ident\u2019-is-missing-in-\u2018qualid\u2019","The field \u2018ident\u2019 is missing in \u2018qualid\u2019"],[72,0,1,"coq:exn.The-recursive-argument-must-be-specified","The recursive argument must be specified"],[55,0,1,"coq:exn.The-reference-X-was-not-found-in-the-current-environment","The reference X was not found in the current environment"],[64,0,1,"coq:exn.The-reference-is-not-unfoldable","The reference is not unfoldable"],[64,0,1,"coq:exn.The-reference-\u2018qualid\u2019-was-not-found-in-the-current-environment","The reference \u2018qualid\u2019 was not found in the current environment"],[58,0,1,"coq:exn.The-term-\"\u2018type\u2019\"-has-type-\"\u2018type\u2019\"-which-should-be-Set,-Prop-or-Type","The term "\u2018type\u2019" has type "\u2018type\u2019" which should be Set, Prop or Type"],[2,0,1,"coq:exn.The-term-\u2018qualid\u2019-is-already-defined-as-foreign-custom-constant","The term \u2018qualid\u2019 is already defined as foreign custom constant"],[2,0,1,"coq:exn.The-term-\u2018qualid\u2019-is-already-defined-as-inline-custom-constant","The term \u2018qualid\u2019 is already defined as inline custom constant"],[32,0,1,"coq:exn.The-term-\u2018term\u2019-has-type-\u2018type\u2019-which-should-be-Set,-Prop-or-Type","The term \u2018term\u2019 has type \u2018type\u2019 which should be Set, Prop or Type"],[32,0,1,"coq:exn.The-term-\u2018term\u2019-has-type-\u2018type\u2019-while-it-is-expected-to-have-type-\u2018type\u2019'","The term \u2018term\u2019 has type \u2018type\u2019 while it is expected to have type \u2018type\u2019'"],[67,0,1,"coq:exn.The-type-has-no-constructors","The type has no constructors"],[59,0,1,"coq:exn.The-type-\u2018ident\u2019-must-be-registered-before-this-construction-can-be-typechecked","The type \u2018ident\u2019 must be registered before this construction can be typechecked"],[46,0,1,"coq:exn.The-variable-ident-is-bound-several-times-in-pattern-term","The variable ident is bound several times in pattern term"],[58,0,1,"coq:exn.The-variable-\u2018ident\u2019-is-already-declared","The variable \u2018ident\u2019 is already declared"],[40,0,1,"coq:exn.The-\u2018natural\u2019-th-argument-of-\u2018ident\u2019-must-be-\u2018ident\u2019-in-\u2018type\u2019","The \u2018natural\u2019 th argument of \u2018ident\u2019 must be \u2018ident\u2019 in \u2018type\u2019"],[32,3,1,"coq:cmd.Theorem","Theorem"],[54,0,1,"coq:exn.There-is-already-an-Ltac-named-\u2018qualid\u2019","There is already an Ltac named \u2018qualid\u2019"],[54,0,1,"coq:exn.There-is-no-Ltac-named-\u2018qualid\u2019","There is no Ltac named \u2018qualid\u2019"],[29,2,1,"coq:warn.There-is-no-flag-or-option-with-this-name:-\"\u2018setting_name\u2019\"","There is no flag or option with this name: "\u2018setting_name\u2019""],[29,0,1,"coq:exn.There-is-no-flag,-option-or-table-with-this-name:-\"\u2018setting_name\u2019\"","There is no flag, option or table with this name: "\u2018setting_name\u2019""],[29,0,1,"coq:exn.There-is-no-qualid-valued-table-with-this-name:-\"\u2018setting_name\u2019\"","There is no qualid-valued table with this name: "\u2018setting_name\u2019""],[29,0,1,"coq:exn.There-is-no-string-valued-table-with-this-name:-\"\u2018setting_name\u2019\"","There is no string-valued table with this name: "\u2018setting_name\u2019""],[38,0,1,"coq:exn.There-is-nothing-to-end","There is nothing to end"],[29,2,1,"coq:warn.This-command-does-not-support-this-attribute","This command does not support this attribute"],[59,0,1,"coq:exn.This-object-does-not-support-universe-names","This object does not support universe names"],[66,0,1,"coq:exn.This-proof-is-focused,-but-cannot-be-unfocused-this-way","This proof is focused, but cannot be unfocused this way"],[54,0,1,"coq:exn.This-tactic-has-more-than-one-success","This tactic has more than one success"],[59,3,1,"coq:cmd.Time","Time"],[59,3,1,"coq:cmd.Timeout","Timeout"],[71,2,1,"coq:warn.To-avoid-stack-overflow,-large-numbers-in-\u2018type\u2019-are-interpreted-as-applications-of-\u2018qualid\u2019","To avoid stack overflow, large numbers in \u2018type\u2019 are interpreted as applications of \u2018qualid\u2019"],[41,0,1,"coq:exn.To-rename-arguments-the-'rename'-flag-must-be-specified","To rename arguments the 'rename' flag must be specified"],[64,3,1,"coq:cmd.Transparent","Transparent"],[9,4,1,"coq:flag.Transparent-Obligations","Transparent Obligations"],[35,2,1,"coq:warn.Trying-to-mask-the-absolute-name-\u2018qualid\u2019!","Trying to mask the absolute name \u2018qualid\u2019!"],[59,3,1,"coq:cmd.Type","Type"],[67,0,1,"coq:exn.Type-of-\u2018ident\u2019-is-not-an-equality-of-recognized-\u03a3-types:-expected-one-of-sig-sig2-sigT-sigT2-sigT2-ex-or-ex2-but-got-\u2018term\u2019","Type of \u2018ident\u2019 is not an equality of recognized \u03a3 types: expected one of sig sig2 sigT sigT2 sigT2 ex or ex2 but got \u2018term\u2019"],[13,4,1,"coq:flag.Typeclass-Resolution-For-Conversion","Typeclass Resolution For Conversion"],[13,4,1,"coq:flag.Typeclasses-Debug","Typeclasses Debug"],[13,6,1,"coq:opt.Typeclasses-Debug-Verbosity","Typeclasses Debug Verbosity"],[13,6,1,"coq:opt.Typeclasses-Default-Mode","Typeclasses Default Mode"],[13,4,1,"coq:flag.Typeclasses-Dependency-Order","Typeclasses Dependency Order"],[13,6,1,"coq:opt.Typeclasses-Depth","Typeclasses Depth"],[13,4,1,"coq:flag.Typeclasses-Iterative-Deepening","Typeclasses Iterative Deepening"],[13,4,1,"coq:flag.Typeclasses-Limit-Intros","Typeclasses Limit Intros"],[13,3,1,"coq:cmd.Typeclasses-Opaque","Typeclasses Opaque"],[13,4,1,"coq:flag.Typeclasses-Strict-Resolution","Typeclasses Strict Resolution"],[13,3,1,"coq:cmd.Typeclasses-Transparent","Typeclasses Transparent"],[13,4,1,"coq:flag.Typeclasses-Unique-Instances","Typeclasses Unique Instances"],[13,4,1,"coq:flag.Typeclasses-Unique-Solutions","Typeclasses Unique Solutions"],[13,3,1,"coq:cmd.Typeclasses-eauto","Typeclasses eauto"],[67,0,1,"coq:exn.Unable-to-find-an-instance-for-the-variables-\u2018ident\u2019-\u2026-\u2018ident\u2019","Unable to find an instance for the variables \u2018ident\u2019 \u2026 \u2018ident\u2019"],[58,0,1,"coq:exn.Unable-to-find-an-instance-for-the-variables-\u2018ident\u2019\u2026\u2018ident\u2019","Unable to find an instance for the variables \u2018ident\u2019\u2026\u2018ident\u2019"],[46,0,1,"coq:exn.Unable-to-infer-a-match-predicate","Unable to infer a match predicate"],[3,0,1,"coq:exn.Unable-to-satisfy-the-rewriting-constraints","Unable to satisfy the rewriting constraints"],[58,0,1,"coq:exn.Unable-to-unify-\u2018one_term\u2019-with-\u2018one_term\u2019","Unable to unify \u2018one_term\u2019 with \u2018one_term\u2019"],[55,0,1,"coq:exn.Unbound-[value|constructor]-X","Unbound [value|constructor] X"],[54,0,1,"coq:exn.Unbound-context-identifier-\u2018ident\u2019","Unbound context identifier \u2018ident\u2019"],[14,0,1,"coq:exn.Undeclared-universe-\u2018ident\u2019","Undeclared universe \u2018ident\u2019"],[71,3,1,"coq:cmd.Undelimit-Scope","Undelimit Scope"],[66,3,1,"coq:cmd.Undo","Undo"],[71,0,1,"coq:exn.Unexpected-non-option-term-\u2018term\u2019-while-parsing-a-number-notation","Unexpected non-option term \u2018term\u2019 while parsing a number notation"],[71,0,1,"coq:exn.Unexpected-non-option-term-\u2018term\u2019-while-parsing-a-string-notation","Unexpected non-option term \u2018term\u2019 while parsing a string notation"],[71,0,1,"coq:exn.Unexpected-only-parsing-for-an-only-printing-notation","Unexpected only parsing for an only printing notation"],[71,0,1,"coq:exn.Unexpected-only-printing-for-an-only-parsing-notation","Unexpected only printing for an only parsing notation"],[71,0,1,"coq:exn.Unexpected-term-\u2018term\u2019-while-parsing-a-number-notation","Unexpected term \u2018term\u2019 while parsing a number notation"],[71,0,1,"coq:exn.Unexpected-term-\u2018term\u2019-while-parsing-a-string-notation","Unexpected term \u2018term\u2019 while parsing a string notation"],[66,3,1,"coq:cmd.Unfocus","Unfocus"],[66,3,1,"coq:cmd.Unfocused","Unfocused"],[34,4,1,"coq:flag.Uniform-Inductive-Parameters","Uniform Inductive Parameters"],[14,3,1,"coq:cmd.Universe","Universe"],[59,4,1,"coq:flag.Universe-Checking","Universe Checking"],[14,4,1,"coq:flag.Universe-Minimization-ToSet","Universe Minimization ToSet"],[14,4,1,"coq:flag.Universe-Polymorphism","Universe Polymorphism"],[14,0,1,"coq:exn.Universe-inconsistency","Universe inconsistency"],[59,0,1,"coq:exn.Universe-instance-length-is-\u2018natural\u2019-but-should-be-\u2018natural\u2019","Universe instance length is \u2018natural\u2019 but should be \u2018natural\u2019"],[14,3,1,"coq:cmd.Universes","Universes"],[71,0,1,"coq:exn.Unknown-custom-entry","Unknown custom entry"],[71,0,1,"coq:exn.Unknown-custom-entry:-\u2018ident\u2019","Unknown custom entry: \u2018ident\u2019"],[66,0,1,"coq:exn.Unknown-inductive-type","Unknown inductive type"],[29,3,1,"coq:cmd.Unset","Unset"],[66,3,1,"coq:cmd.Unshelve","Unshelve"],[71,0,1,"coq:exn.Unterminated-string-in-notation","Unterminated string in notation"],[28,2,1,"coq:warn.Use-of-\"Variable\"-or-\"Hypothesis\"-outside-sections-behaves-as-\"#[local]-Parameter\"-or-\"#[local]-Axiom\"","Use of "Variable" or "Hypothesis" outside sections behaves as "#[local] Parameter" or "#[local] Axiom""],[71,2,1,"coq:warn.Use-of-\u2018string\u2019-Notation-is-deprecated-as-it-is-inconsistent-with-pattern-syntax","Use of \u2018string\u2019 Notation is deprecated as it is inconsistent with pattern syntax"],[13,2,1,"coq:warn.Using-inferred-default-mode:-\u201cmode\u201d-for-\u201c\u2018ident\u2019\u201d","Using inferred default mode: \u201cmode\u201d for \u201c\u2018ident\u2019\u201d"],[66,3,1,"coq:cmd.Validate-Proof","Validate Proof"],[28,3,1,"coq:cmd.Variable","Variable"],[66,2,1,"coq:warn.Variable-All-is-shadowed-by-Collection-named-All-containing-all-variables","Variable All is shadowed by Collection named All containing all variables"],[28,3,1,"coq:cmd.Variables","Variables"],[40,3,1,"coq:cmd.Variant","Variant"],[59,6,1,"coq:opt.Warnings","Warnings"],[44,0,1,"coq:exn.Wrong-argument-name","Wrong argument name"],[44,0,1,"coq:exn.Wrong-argument-position","Wrong argument position"],[66,0,1,"coq:exn.Wrong-bullet-\u2018bullet\u2019:-Bullet-\u2018bullet\u2019-is-mandatory-here","Wrong bullet \u2018bullet\u2019: Bullet \u2018bullet\u2019 is mandatory here"],[66,0,1,"coq:exn.Wrong-bullet-\u2018bullet\u2019:-Current-bullet-\u2018bullet\u2019-is-not-finished","Wrong bullet \u2018bullet\u2019: Current bullet \u2018bullet\u2019 is not finished"],[54,1,1,"coq:tacn.[-\u2026-|-\u2026-|-\u2026-]-(dispatch)","[ \u2026 | \u2026 | \u2026 ] (dispatch)"],[54,1,1,"coq:tacn.[>-\u2026-|-\u2026-|-\u2026-]-(dispatch)","[> \u2026 | \u2026 | \u2026 ] (dispatch)"],[55,7,1,"coq:attr.abstract","abstract"],[66,1,1,"coq:tacn.abstract","abstract"],[57,1,1,"coq:tacn.abstract-(ssreflect)","abstract (ssreflect)"],[58,1,1,"coq:tacn.absurd","absurd"],[71,7,1,"coq:attr.add_bottom","add_bottom"],[71,7,1,"coq:attr.add_top","add_top"],[66,1,1,"coq:tacn.admit","admit"],[58,1,1,"coq:tacn.apply","apply"],[57,1,1,"coq:tacn.apply-(ssreflect)","apply (ssreflect)"],[58,1,1,"coq:tacn.assert","assert"],[54,1,1,"coq:tacn.assert_fails","assert_fails"],[54,1,1,"coq:tacn.assert_succeeds","assert_succeeds"],[58,1,1,"coq:tacn.assumption","assumption"],[60,1,1,"coq:tacn.auto","auto"],[13,1,1,"coq:tacn.autoapply","autoapply"],[34,2,1,"coq:warn.automatic-prop-lowering","automatic-prop-lowering"],[60,1,1,"coq:tacn.autorewrite","autorewrite"],[60,1,1,"coq:tacn.autounfold","autounfold"],[60,1,1,"coq:tacn.autounfold_one","autounfold_one"],[62,1,1,"coq:tacn.btauto","btauto"],[66,1,1,"coq:tacn.bullet-(--+-*)","bullet (- + *)"],[57,1,1,"coq:tacn.by","by"],[59,7,1,"coq:attr.bypass_check(guard)","bypass_check(guard)"],[59,7,1,"coq:attr.bypass_check(positivity)","bypass_check(positivity)"],[59,7,1,"coq:attr.bypass_check(universes)","bypass_check(universes)"],[42,7,1,"coq:attr.canonical","canonical"],[67,1,1,"coq:tacn.case","case"],[57,1,1,"coq:tacn.case-(ssreflect)","case (ssreflect)"],[67,1,1,"coq:tacn.case_eq","case_eq"],[64,1,1,"coq:tacn.cbn","cbn"],[64,1,1,"coq:tacn.cbv","cbv"],[64,1,1,"coq:tacn.change","change"],[64,1,1,"coq:tacn.change_no_check","change_no_check"],[58,1,1,"coq:tacn.classical_left","classical_left"],[58,1,1,"coq:tacn.classical_right","classical_right"],[58,1,1,"coq:tacn.clear","clear"],[58,1,1,"coq:tacn.clear-dependent","clear dependent"],[38,7,1,"coq:attr.clearbody","clearbody"],[58,1,1,"coq:tacn.clearbody","clearbody"],[71,2,1,"coq:warn.closed-notation-not-level-0","closed-notation-not-level-0"],[67,1,1,"coq:tacn.cofix","cofix"],[67,1,1,"coq:tacn.compare","compare"],[64,1,1,"coq:tacn.compute","compute"],[57,1,1,"coq:tacn.congr","congr"],[62,1,1,"coq:tacn.congruence","congruence"],[54,1,1,"coq:tacn.constr_eq","constr_eq"],[54,1,1,"coq:tacn.constr_eq_nounivs","constr_eq_nounivs"],[54,1,1,"coq:tacn.constr_eq_strict","constr_eq_strict"],[67,1,1,"coq:tacn.constructor","constructor"],[54,1,1,"coq:tacn.context","context"],[58,1,1,"coq:tacn.contradict","contradict"],[58,1,1,"coq:tacn.contradiction","contradiction"],[54,1,1,"coq:tacn.convert","convert"],[58,1,1,"coq:tacn.cut","cut"],[66,1,1,"coq:tacn.cycle","cycle"],[60,1,1,"coq:tacn.debug-auto","debug auto"],[60,1,1,"coq:tacn.debug-eauto","debug eauto"],[60,1,1,"coq:tacn.debug-trivial","debug trivial"],[67,1,1,"coq:tacn.decide","decide"],[67,1,1,"coq:tacn.decide-equality","decide equality"],[67,1,1,"coq:tacn.decompose","decompose"],[67,1,1,"coq:tacn.decompose-record","decompose record"],[67,1,1,"coq:tacn.decompose-sum","decompose sum"],[67,1,1,"coq:tacn.dependent-destruction","dependent destruction"],[58,1,1,"coq:tacn.dependent-generalize_eqs","dependent generalize_eqs"],[58,1,1,"coq:tacn.dependent-generalize_eqs_vars","dependent generalize_eqs_vars"],[67,1,1,"coq:tacn.dependent-induction","dependent induction"],[67,1,1,"coq:tacn.dependent-inversion","dependent inversion"],[67,1,1,"coq:tacn.dependent-inversion_clear","dependent inversion_clear"],[67,1,1,"coq:tacn.dependent-rewrite","dependent rewrite"],[67,1,1,"coq:tacn.dependent-simple-inversion","dependent simple inversion"],[74,7,1,"coq:attr.deprecated","deprecated"],[67,1,1,"coq:tacn.destauto","destauto"],[67,1,1,"coq:tacn.destruct","destruct"],[60,1,1,"coq:tacn.dfs-eauto","dfs eauto"],[62,1,1,"coq:tacn.dintuition","dintuition"],[27,1,1,"coq:tacn.discrR","discrR"],[67,1,1,"coq:tacn.discriminate","discriminate"],[54,1,1,"coq:tacn.do","do"],[57,1,1,"coq:tacn.do-(ssreflect)","do (ssreflect)"],[57,1,1,"coq:tacn.done","done"],[62,1,1,"coq:tacn.dtauto","dtauto"],[58,1,1,"coq:tacn.eapply","eapply"],[58,1,1,"coq:tacn.eassert","eassert"],[58,1,1,"coq:tacn.eassumption","eassumption"],[60,1,1,"coq:tacn.easy","easy"],[60,1,1,"coq:tacn.eauto","eauto"],[67,1,1,"coq:tacn.ecase","ecase"],[67,1,1,"coq:tacn.econstructor","econstructor"],[67,1,1,"coq:tacn.edestruct","edestruct"],[67,1,1,"coq:tacn.ediscriminate","ediscriminate"],[67,1,1,"coq:tacn.eelim","eelim"],[58,1,1,"coq:tacn.eenough","eenough"],[58,1,1,"coq:tacn.eexact","eexact"],[67,1,1,"coq:tacn.eexists","eexists"],[67,1,1,"coq:tacn.einduction","einduction"],[67,1,1,"coq:tacn.einjection","einjection"],[58,1,1,"coq:tacn.eintros","eintros"],[67,1,1,"coq:tacn.eleft","eleft"],[67,1,1,"coq:tacn.elim","elim"],[57,1,1,"coq:tacn.elim-(ssreflect)","elim (ssreflect)"],[58,1,1,"coq:tacn.enough","enough"],[58,1,1,"coq:tacn.epose","epose"],[58,1,1,"coq:tacn.epose-proof","epose proof"],[58,1,1,"coq:tacn.eremember","eremember"],[64,1,1,"coq:tacn.erewrite","erewrite"],[67,1,1,"coq:tacn.eright","eright"],[58,1,1,"coq:tacn.eset","eset"],[67,1,1,"coq:tacn.esimplify_eq","esimplify_eq"],[67,1,1,"coq:tacn.esplit","esplit"],[64,1,1,"coq:tacn.etransitivity","etransitivity"],[64,1,1,"coq:tacn.eval","eval"],[58,1,1,"coq:tacn.evar","evar"],[58,1,1,"coq:tacn.exact","exact"],[57,1,1,"coq:tacn.exact-(ssreflect)","exact (ssreflect)"],[58,1,1,"coq:tacn.exact_no_check","exact_no_check"],[54,1,1,"coq:tacn.exactly_once","exactly_once"],[58,1,1,"coq:tacn.exfalso","exfalso"],[67,1,1,"coq:tacn.exists","exists"],[35,7,1,"coq:attr.export","export"],[64,1,1,"coq:tacn.f_equal","f_equal"],[54,1,1,"coq:tacn.fail","fail"],[11,1,1,"coq:tacn.field","field"],[11,1,1,"coq:tacn.field_lookup","field_lookup"],[11,1,1,"coq:tacn.field_simplify","field_simplify"],[11,1,1,"coq:tacn.field_simplify_eq","field_simplify_eq"],[54,1,1,"coq:tacn.finish_timing","finish_timing"],[54,1,1,"coq:tacn.first","first"],[57,1,1,"coq:tacn.first-(ssreflect)","first (ssreflect)"],[57,9,1,"coq:tacv.first-last","first last"],[62,1,1,"coq:tacn.firstorder","firstorder"],[67,1,1,"coq:tacn.fix","fix"],[64,1,1,"coq:tacn.fold","fold"],[54,1,1,"coq:tacn.fresh","fresh"],[54,1,1,"coq:tacn.fun","fun"],[72,1,1,"coq:tacn.functional-induction","functional induction"],[72,1,1,"coq:tacn.functional-inversion","functional inversion"],[58,1,1,"coq:tacn.generalize","generalize"],[58,1,1,"coq:tacn.generalize-dependent","generalize dependent"],[58,1,1,"coq:tacn.generalize_eqs","generalize_eqs"],[58,1,1,"coq:tacn.generalize_eqs_vars","generalize_eqs_vars"],[57,1,1,"coq:tacn.generally-have","generally have"],[54,1,1,"coq:tacn.gfail","gfail"],[66,1,1,"coq:tacn.give_up","give_up"],[35,7,1,"coq:attr.global","global"],[54,1,1,"coq:tacn.guard","guard"],[54,1,1,"coq:tacn.has_evar","has_evar"],[57,1,1,"coq:tacn.have","have"],[3,1,1,"coq:tacn.head_of_constr","head_of_constr"],[64,1,1,"coq:tacn.hnf","hnf"],[54,1,1,"coq:tacn.idtac","idtac"],[55,1,1,"coq:tacn.if-then-else-(Ltac2)","if-then-else (Ltac2)"],[57,1,1,"coq:tacn.in","in"],[67,1,1,"coq:tacn.induction","induction"],[54,3,1,"coq:cmd.infoH","infoH"],[60,1,1,"coq:tacn.info_auto","info_auto"],[60,1,1,"coq:tacn.info_eauto","info_eauto"],[60,1,1,"coq:tacn.info_trivial","info_trivial"],[67,1,1,"coq:tacn.injection","injection"],[58,1,1,"coq:tacn.instantiate","instantiate"],[58,1,1,"coq:tacn.intro","intro"],[58,1,1,"coq:tacn.intros","intros"],[58,1,1,"coq:tacn.intros-until","intros until"],[62,1,1,"coq:tacn.intuition","intuition"],[67,1,1,"coq:tacn.inversion","inversion"],[67,1,1,"coq:tacn.inversion_clear","inversion_clear"],[67,1,1,"coq:tacn.inversion_sigma","inversion_sigma"],[54,1,1,"coq:tacn.is_cofix","is_cofix"],[54,1,1,"coq:tacn.is_const","is_const"],[54,1,1,"coq:tacn.is_constructor","is_constructor"],[54,1,1,"coq:tacn.is_evar","is_evar"],[54,1,1,"coq:tacn.is_fix","is_fix"],[54,1,1,"coq:tacn.is_ground","is_ground"],[54,1,1,"coq:tacn.is_ind","is_ind"],[54,1,1,"coq:tacn.is_proj","is_proj"],[54,1,1,"coq:tacn.is_var","is_var"],[58,1,1,"coq:tacn.lapply","lapply"],[58,0,1,"coq:exn.lapply-needs-a-non-dependent-product","lapply needs a non-dependent product"],[57,1,1,"coq:tacn.last","last"],[57,9,1,"coq:tacv.last-first","last first"],[64,1,1,"coq:tacn.lazy","lazy"],[55,1,1,"coq:tacn.lazy_match!","lazy_match!"],[55,1,1,"coq:tacn.lazy_match!-goal","lazy_match! goal"],[54,1,1,"coq:tacn.lazymatch","lazymatch"],[54,1,1,"coq:tacn.lazymatch-goal","lazymatch goal"],[67,1,1,"coq:tacn.left","left"],[54,1,1,"coq:tacn.let","let"],[5,1,1,"coq:tacn.lia","lia"],[35,7,1,"coq:attr.local","local"],[5,1,1,"coq:tacn.lra","lra"],[54,1,1,"coq:tacn.ltac-seq","ltac-seq"],[54,1,1,"coq:tacn.match","match"],[55,1,1,"coq:tacn.match-(Ltac2)","match (Ltac2)"],[54,1,1,"coq:tacn.match-goal","match goal"],[55,1,1,"coq:tacn.match!","match!"],[55,1,1,"coq:tacn.match!-goal","match! goal"],[13,7,1,"coq:attr.mode","mode"],[58,1,1,"coq:tacn.move","move"],[57,1,1,"coq:tacn.move-(ssreflect)","move (ssreflect)"],[55,1,1,"coq:tacn.multi_match!","multi_match!"],[55,1,1,"coq:tacn.multi_match!-goal","multi_match! goal"],[54,1,1,"coq:tacn.multimatch","multimatch"],[54,1,1,"coq:tacn.multimatch-goal","multimatch goal"],[58,1,1,"coq:tacn.native_cast_no_check","native_cast_no_check"],[64,1,1,"coq:tacn.native_compute","native_compute"],[5,1,1,"coq:tacn.nia","nia"],[4,7,1,"coq:attr.nonuniform","nonuniform"],[54,0,1,"coq:exn.not-a-cofix-definition","not a cofix definition"],[54,0,1,"coq:exn.not-a-constant","not a constant"],[54,0,1,"coq:exn.not-a-constructor","not a constructor"],[54,0,1,"coq:exn.not-a-fix-definition","not a fix definition"],[54,0,1,"coq:exn.not-a-primitive-projection","not a primitive projection"],[54,0,1,"coq:exn.not-an-(co)inductive-datatype","not an (co)inductive datatype"],[54,1,1,"coq:tacn.not_evar","not_evar"],[71,2,1,"coq:warn.notation-incompatible-prefix","notation-incompatible-prefix"],[60,1,1,"coq:tacn.now","now"],[64,1,1,"coq:tacn.now_show","now_show"],[5,1,1,"coq:tacn.nra","nra"],[7,1,1,"coq:tacn.nsatz","nsatz"],[7,1,1,"coq:tacn.nsatz_compute","nsatz_compute"],[54,1,1,"coq:tacn.numgoals","numgoals"],[54,1,1,"coq:tacn.once","once"],[54,1,1,"coq:tacn.only","only"],[54,1,1,"coq:tacn.optimize_heap","optimize_heap"],[57,1,1,"coq:tacn.over","over"],[71,0,1,"coq:exn.overflow-in-int63-literal-\u2018bigint\u2019","overflow in int63 literal \u2018bigint\u2019"],[64,1,1,"coq:tacn.pattern","pattern"],[58,1,1,"coq:tacn.pose","pose"],[57,1,1,"coq:tacn.pose-(ssreflect)","pose (ssreflect)"],[58,1,1,"coq:tacn.pose-proof","pose proof"],[71,2,1,"coq:warn.postfix-notation-not-level-1","postfix-notation-not-level-1"],[40,7,1,"coq:attr.private(matching)","private(matching)"],[9,7,1,"coq:attr.program","program"],[54,1,1,"coq:tacn.progress","progress"],[37,7,1,"coq:attr.projections(primitive)","projections(primitive)"],[11,1,1,"coq:tacn.protect_fv","protect_fv"],[5,1,1,"coq:tacn.psatz","psatz"],[59,0,1,"coq:exn.public-name-according-to-findlib,-for-example","public name according to findlib, for example"],[58,1,1,"coq:tacn.rapply","rapply"],[64,1,1,"coq:tacn.red","red"],[13,7,1,"coq:attr.refine","refine"],[58,1,1,"coq:tacn.refine","refine"],[64,1,1,"coq:tacn.reflexivity","reflexivity"],[58,1,1,"coq:tacn.remember","remember"],[58,1,1,"coq:tacn.rename","rename"],[54,1,1,"coq:tacn.repeat","repeat"],[64,1,1,"coq:tacn.replace","replace"],[54,1,1,"coq:tacn.reset-ltac-profile","reset ltac profile"],[54,1,1,"coq:tacn.restart_timer","restart_timer"],[4,7,1,"coq:attr.reversible","reversible"],[58,1,1,"coq:tacn.revert","revert"],[58,1,1,"coq:tacn.revert-dependent","revert dependent"],[66,1,1,"coq:tacn.revgoals","revgoals"],[64,1,1,"coq:tacn.rewrite","rewrite"],[57,1,1,"coq:tacn.rewrite-(ssreflect)","rewrite (ssreflect)"],[64,1,1,"coq:tacn.rewrite-*","rewrite *"],[3,1,1,"coq:tacn.rewrite_db","rewrite_db"],[3,1,1,"coq:tacn.rewrite_strat","rewrite_strat"],[67,1,1,"coq:tacn.right","right"],[11,1,1,"coq:tacn.ring","ring"],[11,1,1,"coq:tacn.ring_lookup","ring_lookup"],[11,1,1,"coq:tacn.ring_simplify","ring_simplify"],[62,1,1,"coq:tacn.rtauto","rtauto"],[58,1,1,"coq:tacn.set","set"],[57,1,1,"coq:tacn.set-(ssreflect)","set (ssreflect)"],[3,1,1,"coq:tacn.setoid_etransitivity","setoid_etransitivity"],[3,1,1,"coq:tacn.setoid_reflexivity","setoid_reflexivity"],[3,1,1,"coq:tacn.setoid_replace","setoid_replace"],[3,1,1,"coq:tacn.setoid_rewrite","setoid_rewrite"],[3,1,1,"coq:tacn.setoid_symmetry","setoid_symmetry"],[3,1,1,"coq:tacn.setoid_transitivity","setoid_transitivity"],[59,0,1,"coq:exn.shared-library-failed:-Coq-Error:-\u2018string\u2019-is-not-a-valid","shared library failed: Coq Error: \u2018string\u2019 is not a valid"],[66,1,1,"coq:tacn.shelve","shelve"],[66,1,1,"coq:tacn.shelve_unifiable","shelve_unifiable"],[54,1,1,"coq:tacn.show-ltac-profile","show ltac profile"],[64,1,1,"coq:tacn.simpl","simpl"],[58,1,1,"coq:tacn.simple-apply","simple apply"],[62,1,1,"coq:tacn.simple-congruence","simple congruence"],[67,1,1,"coq:tacn.simple-destruct","simple destruct"],[58,1,1,"coq:tacn.simple-eapply","simple eapply"],[67,1,1,"coq:tacn.simple-induction","simple induction"],[67,1,1,"coq:tacn.simple-injection","simple injection"],[67,1,1,"coq:tacn.simple-inversion","simple inversion"],[64,1,1,"coq:tacn.simple-subst","simple subst"],[67,1,1,"coq:tacn.simplify_eq","simplify_eq"],[72,1,1,"coq:tacn.soft-functional-induction","soft functional induction"],[54,1,1,"coq:tacn.solve","solve"],[66,1,1,"coq:tacn.solve_constraints","solve_constraints"],[58,1,1,"coq:tacn.specialize","specialize"],[58,1,1,"coq:tacn.specialize_eqs","specialize_eqs"],[67,1,1,"coq:tacn.split","split"],[27,1,1,"coq:tacn.split_Rabs","split_Rabs"],[27,1,1,"coq:tacn.split_Rmult","split_Rmult"],[54,1,1,"coq:tacn.start-ltac-profiling","start ltac profiling"],[64,1,1,"coq:tacn.stepl","stepl"],[64,1,1,"coq:tacn.stepr","stepr"],[54,1,1,"coq:tacn.stop-ltac-profiling","stop ltac profiling"],[64,1,1,"coq:tacn.subst","subst"],[64,1,1,"coq:tacn.substitute","substitute"],[57,1,1,"coq:tacn.suff","suff"],[57,1,1,"coq:tacn.suffices","suffices"],[66,1,1,"coq:tacn.swap","swap"],[64,1,1,"coq:tacn.symmetry","symmetry"],[62,1,1,"coq:tacn.tauto","tauto"],[34,0,1,"coq:exn.template-and-polymorphism-not-compatible","template and polymorphism not compatible"],[54,1,1,"coq:tacn.time","time"],[54,1,1,"coq:tacn.time_constr","time_constr"],[54,1,1,"coq:tacn.timeout","timeout"],[64,1,1,"coq:tacn.transitivity","transitivity"],[66,1,1,"coq:tacn.transparent_abstract","transparent_abstract"],[60,1,1,"coq:tacn.trivial","trivial"],[54,1,1,"coq:tacn.try","try"],[54,1,1,"coq:tacn.tryif","tryif"],[54,1,1,"coq:tacn.type-of","type of"],[54,1,1,"coq:tacn.type_term","type_term"],[13,1,1,"coq:tacn.typeclasses-eauto","typeclasses eauto"],[57,1,1,"coq:tacn.under","under"],[64,1,1,"coq:tacn.unfold","unfold"],[54,1,1,"coq:tacn.unify","unify"],[14,7,1,"coq:attr.universes(cumulative)","universes(cumulative)"],[14,7,1,"coq:attr.universes(polymorphic)","universes(polymorphic)"],[34,7,1,"coq:attr.universes(template)","universes(template)"],[57,1,1,"coq:tacn.unlock","unlock"],[66,1,1,"coq:tacn.unshelve","unshelve"],[66,7,1,"coq:attr.using","using"],[58,1,1,"coq:tacn.vm_cast_no_check","vm_cast_no_check"],[64,1,1,"coq:tacn.vm_compute","vm_compute"],[74,7,1,"coq:attr.warn","warn"],[29,7,1,"coq:attr.warning","warning"],[29,7,1,"coq:attr.warnings","warnings"],[64,1,1,"coq:tacn.with_strategy","with_strategy"],[57,1,1,"coq:tacn.without-loss","without loss"],[5,1,1,"coq:tacn.wlia","wlia"],[57,1,1,"coq:tacn.wlog","wlog"],[5,1,1,"coq:tacn.wlra_Q","wlra_Q"],[5,1,1,"coq:tacn.wnia","wnia"],[5,1,1,"coq:tacn.wnra_Q","wnra_Q"],[5,1,1,"coq:tacn.wpsatz_Q","wpsatz_Q"],[5,1,1,"coq:tacn.wpsatz_Z","wpsatz_Z"],[5,1,1,"coq:tacn.wsos_Q","wsos_Q"],[5,1,1,"coq:tacn.wsos_Z","wsos_Z"],[5,1,1,"coq:tacn.xlia","xlia"],[5,1,1,"coq:tacn.xlra_Q","xlra_Q"],[5,1,1,"coq:tacn.xlra_R","xlra_R"],[5,1,1,"coq:tacn.xnia","xnia"],[5,1,1,"coq:tacn.xnra_Q","xnra_Q"],[5,1,1,"coq:tacn.xnra_R","xnra_R"],[5,1,1,"coq:tacn.xpsatz_Q","xpsatz_Q"],[5,1,1,"coq:tacn.xpsatz_R","xpsatz_R"],[5,1,1,"coq:tacn.xpsatz_Z","xpsatz_Z"],[5,1,1,"coq:tacn.xsos_Q","xsos_Q"],[5,1,1,"coq:tacn.xsos_R","xsos_R"],[5,1,1,"coq:tacn.xsos_Z","xsos_Z"],[5,1,1,"coq:tacn.zify","zify"],[5,1,1,"coq:tacn.zify_elim_let","zify_elim_let"],[5,1,1,"coq:tacn.zify_iter_let","zify_iter_let"],[5,1,1,"coq:tacn.zify_iter_specs","zify_iter_specs"],[5,1,1,"coq:tacn.zify_op","zify_op"],[5,1,1,"coq:tacn.zify_saturate","zify_saturate"],[66,1,1,"coq:tacn.{","{"],[54,1,1,"coq:tacn.||-(first-tactic-making-progress)","|| (first tactic making progress)"],[66,1,1,"coq:tacn.}","}"],[4,0,1,"coq:exn.\u2018coercion_class\u2019-must-be-a-transparent-constant","\u2018coercion_class\u2019 must be a transparent constant"],[37,0,1,"coq:exn.\u2018ident\u2019-already-exists","\u2018ident\u2019 already exists"],[37,2,1,"coq:warn.\u2018ident\u2019-cannot-be-defined","\u2018ident\u2019 cannot be defined"],[37,2,1,"coq:warn.\u2018ident\u2019-cannot-be-defined-because-it-is-informative-and-\u2018ident\u2019-is-not","\u2018ident\u2019 cannot be defined because it is informative and \u2018ident\u2019 is not"],[37,2,1,"coq:warn.\u2018ident\u2019-cannot-be-defined-because-the-projection-\u2018ident\u2019-was-not-defined","\u2018ident\u2019 cannot be defined because the projection \u2018ident\u2019 was not defined"],[13,2,1,"coq:warn.\u2018ident\u2019-is-already-declared-as-a-typeclass","\u2018ident\u2019 is already declared as a typeclass"],[58,0,1,"coq:exn.\u2018ident\u2019-is-already-used","\u2018ident\u2019 is already used"],[66,2,1,"coq:warn.\u2018ident\u2019-is-both-name-of-a-Collection-and-Variable,-Collection-\u2018ident\u2019-takes-precedence-over-Variable","\u2018ident\u2019 is both name of a Collection and Variable, Collection \u2018ident\u2019 takes precedence over Variable"],[58,0,1,"coq:exn.\u2018ident\u2019-is-not-a-local-definition","\u2018ident\u2019 is not a local definition"],[67,0,1,"coq:exn.\u2018ident\u2019-is-not-an-equality-of-\u03a3-types","\u2018ident\u2019 is not an equality of \u03a3 types"],[64,0,1,"coq:exn.\u2018ident\u2019-is-opaque","\u2018ident\u2019 is opaque"],[58,0,1,"coq:exn.\u2018ident\u2019-is-used-in-the-conclusion","\u2018ident\u2019 is used in the conclusion"],[58,0,1,"coq:exn.\u2018ident\u2019-is-used-in-the-hypothesis-\u2018ident\u2019","\u2018ident\u2019 is used in the hypothesis \u2018ident\u2019"],[66,2,1,"coq:warn.\u2018ident\u2019-was-already-a-defined-Variable,-the-name-\u2018ident\u2019-will-refer-to-Collection-when-executing-\"Proof-using\"-command","\u2018ident\u2019 was already a defined Variable, the name \u2018ident\u2019 will refer to Collection when executing "Proof using" command"],[60,0,1,"coq:exn.\u2018qualid\u2019-cannot-be-used-as-a-hint","\u2018qualid\u2019 cannot be used as a hint"],[64,0,1,"coq:exn.\u2018qualid\u2019-does-not-occur","\u2018qualid\u2019 does not occur"],[4,2,1,"coq:warn.\u2018qualid\u2019-does-not-respect-the-uniform-inheritance-condition","\u2018qualid\u2019 does not respect the uniform inheritance condition"],[4,0,1,"coq:exn.\u2018qualid\u2019-is-already-a-coercion","\u2018qualid\u2019 is already a coercion"],[71,0,1,"coq:exn.\u2018qualid\u2019-is-bound-to-a-notation-that-does-not-denote-a-reference","\u2018qualid\u2019 is bound to a notation that does not denote a reference"],[4,0,1,"coq:exn.\u2018qualid\u2019-is-not-a-function","\u2018qualid\u2019 is not a function"],[35,0,1,"coq:exn.\u2018qualid\u2019-is-not-a-module","\u2018qualid\u2019 is not a module"],[60,0,1,"coq:exn.\u2018qualid\u2019-is-not-an-inductive-type","\u2018qualid\u2019 is not an inductive type"],[59,0,1,"coq:exn.\u2018qualid\u2019-not-a-defined-object","\u2018qualid\u2019 not a defined object"],[4,0,1,"coq:exn.\u2018qualid\u2019-not-declared","\u2018qualid\u2019 not declared"],[71,0,1,"coq:exn.\u2018qualid\u2019-was-already-mapped-to-\u2018qualid\u2019-and-cannot-be-remapped-to-\u2018qualid\u2019","\u2018qualid\u2019 was already mapped to \u2018qualid\u2019 and cannot be remapped to \u2018qualid\u2019"],[74,2,1,"coq:warn.\u2018string\u2019","\u2018string\u2019"],[71,0,1,"coq:exn.\u2018type\u2019-is-not-an-inductive-type","\u2018type\u2019 is not an inductive type"],[71,2,1,"coq:warn.\u2018type\u2019-was-already-mapped-to-\u2018type\u2019,-mapping-it-also-to-\u2018type\u2019-might-yield-ill-typed-terms-when-using-the-notation","\u2018type\u2019 was already mapped to \u2018type\u2019, mapping it also to \u2018type\u2019 might yield ill typed terms when using the notation"],[54,1,1,"coq:tacn.\u2026-:-\u2026-(goal-selector)","\u2026 : \u2026 (goal selector)"],[57,1,1,"coq:tacn.\u2026-:-\u2026-(ssreflect)","\u2026 : \u2026 (ssreflect)"]],""All" is a predefined collection containing all variables":[[66,0,1,"coq:exn.\"All\"-is-a-predefined-collection-containing-all-variables.-It-can't-be-redefined"," It can't be redefined"]],"..":[[4,2,1,"coq:warn....-is-not-definitionally-an-identity-function"," is not definitionally an identity function"]],"Argument \u2018name\u2019 is a trailing implicit, so it can't be declared non maximal":[[44,0,1,"coq:exn.Argument-\u2018name\u2019-is-a-trailing-implicit,-so-it-can't-be-declared-non-maximal.-Please-use-{-}-instead-of-[-]"," Please use { } instead of [ ]"]],"Cannot infer a term for this placeholder":[[44,0,1,"coq:exn.Cannot-infer-a-term-for-this-placeholder.-(Casual-use-of-implicit-arguments)"," (Casual use of implicit arguments)"],[58,0,1,"coq:exn.Cannot-infer-a-term-for-this-placeholder.-(refine)"," (refine)"]],"Compiled library \u2018ident\u2019":[[59,0,1,"coq:exn.Compiled-library-\u2018ident\u2019.vo-makes-inconsistent-assumptions-over-library-\u2018qualid\u2019","vo makes inconsistent assumptions over library \u2018qualid\u2019"]],"Duplicate clear of H":[[57,2,1,"coq:warn.Duplicate-clear-of-H.-Use-{-}H-instead-of-{-H-}H"," Use { }H instead of { H }H"]],"File ... found twice in ..":[[59,2,1,"coq:warn.File-...-found-twice-in-...",""]],"Goal is solvable by congruence but some arguments are missing":[[62,0,1,"coq:exn.Goal-is-solvable-by-congruence-but-some-arguments-are-missing.-Try-congruence-with-\u2018term\u2019\u2026\u2018term\u2019,-replacing-metavariables-by-arbitrary-terms"," Try congruence with \u2018term\u2019\u2026\u2018term\u2019, replacing metavariables by arbitrary terms"]],"Library File (transitively required) \u2018qualid\u2019 is deprecated since \u2018string\u2019. \u2018string\u2019":[[74,2,1,"coq:warn.Library-File-(transitively-required)-\u2018qualid\u2019-is-deprecated-since-\u2018string\u2019.-\u2018string\u2019.-Use-\u2018qualid\u2019-instead"," Use \u2018qualid\u2019 instead"]],"Library File \u2018qualid\u2019 is deprecated since \u2018string\u2019. \u2018string\u2019":[[74,2,1,"coq:warn.Library-File-\u2018qualid\u2019-is-deprecated-since-\u2018string\u2019.-\u2018string\u2019.-Use-\u2018qualid\u2019-instead"," Use \u2018qualid\u2019 instead"]],"Ltac Profiler encountered an invalid stack (no self node)":[[54,2,1,"coq:warn.Ltac-Profiler-encountered-an-invalid-stack-(no-self-node).-This-can-happen-if-you-reset-the-profile-during-tactic-execution"," This can happen if you reset the profile during tactic execution"]],"Ltac2 alias \u2018qualid\u2019 is deprecated since \u2018string\u2019":[[74,2,1,"coq:warn.Ltac2-alias-\u2018qualid\u2019-is-deprecated-since-\u2018string\u2019.-\u2018string\u2019"," \u2018string\u2019"]],"Ltac2 constructor \u2018qualid\u2019 is deprecated since \u2018string\u2019":[[74,2,1,"coq:warn.Ltac2-constructor-\u2018qualid\u2019-is-deprecated-since-\u2018string\u2019.-\u2018string\u2019"," \u2018string\u2019"]],"Ltac2 definition \u2018qualid\u2019 is deprecated since \u2018string\u2019":[[74,2,1,"coq:warn.Ltac2-definition-\u2018qualid\u2019-is-deprecated-since-\u2018string\u2019.-\u2018string\u2019"," \u2018string\u2019"]],"Ltac2 notation \u2018ltac2_scope\u2019\u2026\u2018ltac2_scope\u2019 is deprecated since \u2018string\u2019":[[74,2,1,"coq:warn.Ltac2-notation-\u2018ltac2_scope\u2019\u2026\u2018ltac2_scope\u2019-is-deprecated-since-\u2018string\u2019.-\u2018string\u2019"," \u2018string\u2019"]],"Nested proofs are discouraged and not allowed by default. This error probably means that you forgot to close the last "Proof." with "Qed." or "Defined."":[[32,0,1,"coq:exn.Nested-proofs-are-discouraged-and-not-allowed-by-default.-This-error-probably-means-that-you-forgot-to-close-the-last-\"Proof.\"-with-\"Qed.\"-or-\"Defined.\".-If-you-really-intended-to-use-nested-proofs,-you-can-do-so-by-turning-the-\"Nested-Proofs-Allowed\"-flag-on"," If you really intended to use nested proofs, you can do so by turning the "Nested Proofs Allowed" flag on"]],"New coercion path ... is ambiguous with existing ..":[[4,2,1,"coq:warn.New-coercion-path-...-is-ambiguous-with-existing-...",""]],"No information can be deduced from this equality and the injectivity of constructors. This may be because the terms are convertible, or due to pattern matching restrictions in the sort Prop":[[67,0,1,"coq:exn.No-information-can-be-deduced-from-this-equality-and-the-injectivity-of-constructors.-This-may-be-because-the-terms-are-convertible,-or-due-to-pattern-matching-restrictions-in-the-sort-Prop.-You-can-try-to-use-option-Set-Keep-Proof-Equalities"," You can try to use option Set Keep Proof Equalities"]],"No such bound variable \u2018ident\u2019 (possible names are: \u2018ident\u2019 ..":[[58,0,1,"coq:exn.No-such-bound-variable-\u2018ident\u2019-(possible-names-are:-\u2018ident\u2019-...)",")"]],"No such goal":[[54,0,1,"coq:exn.No-such-goal.-(Goal-selector)"," (Goal selector)"],[54,0,1,"coq:exn.No-such-goal.-(fail)"," (fail)"],[66,0,1,"coq:exn.No-such-goal.-Focus-next-goal-with-bullet-\u2018bullet\u2019"," Focus next goal with bullet \u2018bullet\u2019"],[66,0,1,"coq:exn.No-such-goal.-Try-unfocusing-with-}"," Try unfocusing with }"]],"Notation \u2018string\u2019 is deprecated since \u2018string\u2019. \u2018string\u2019":[[74,2,1,"coq:warn.Notation-\u2018string\u2019-is-deprecated-since-\u2018string\u2019.-\u2018string\u2019.-Use-\u2018qualid\u2019-instead"," Use \u2018qualid\u2019 instead"]],"Proof is not complete":[[66,0,1,"coq:exn.Proof-is-not-complete.-(abstract)"," (abstract)"],[58,0,1,"coq:exn.Proof-is-not-complete.-(assert)"," (assert)"]],"Require inside a module is deprecated and strongly discouraged":[[59,2,1,"coq:warn.Require-inside-a-module-is-deprecated-and-strongly-discouraged.-You-can-Require-a-module-at-toplevel-and-optionally-Import-it-inside-another-one"," You can Require a module at toplevel and optionally Import it inside another one"]],"Required library \u2018qualid\u2019 matches several files in path (found file.vo, file.vo, ..":[[59,0,1,"coq:exn.Required-library-\u2018qualid\u2019-matches-several-files-in-path-(found-file.vo,-file.vo,-...)",")"]],"SSReflect: cannot obtain new equations out of ..":[[57,2,1,"coq:warn.SSReflect:-cannot-obtain-new-equations-out-of-...",""]],"Tactic Notation \u2018qualid\u2019 is deprecated since \u2018string\u2019":[[74,2,1,"coq:warn.Tactic-Notation-\u2018qualid\u2019-is-deprecated-since-\u2018string\u2019.-\u2018string\u2019"," \u2018string\u2019"]],"Tactic \u2018qualid\u2019 is deprecated since \u2018string\u2019":[[74,2,1,"coq:warn.Tactic-\u2018qualid\u2019-is-deprecated-since-\u2018string\u2019.-\u2018string\u2019"," \u2018string\u2019"]],"The constant \u2018number\u2019 is not a binary64 floating-point value. A closest value \u2018number\u2019 will be used and unambiguously printed \u2018number\u2019":[[27,2,1,"coq:warn.The-constant-\u2018number\u2019-is-not-a-binary64-floating-point-value.-A-closest-value-\u2018number\u2019-will-be-used-and-unambiguously-printed-\u2018number\u2019.-[inexact-float,parsing]"," [inexact-float,parsing]"]],"The file \u2018ident\u2019":[[59,0,1,"coq:exn.The-file-\u2018ident\u2019.vo-contains-library-\u2018qualid\u2019-and-not-library-\u2018qualid\u2019","vo contains library \u2018qualid\u2019 and not library \u2018qualid\u2019"]],"The relation \u2018ident\u2019 is not a declared reflexive relation. Maybe you need to require the Stdlib.Classes":[[64,0,1,"coq:exn.The-relation-\u2018ident\u2019-is-not-a-declared-reflexive-relation.-Maybe-you-need-to-require-the-Stdlib.Classes.RelationClasses-library","RelationClasses library"]],"The relation \u2018ident\u2019 is not a declared symmetric relation. Maybe you need to require the Stdlib.Classes":[[64,0,1,"coq:exn.The-relation-\u2018ident\u2019-is-not-a-declared-symmetric-relation.-Maybe-you-need-to-require-the-Stdlib.Classes.RelationClasses-library","RelationClasses library"]],"The relation \u2018ident\u2019 is not a declared transitive relation. Maybe you need to require the Stdlib.Classes":[[64,0,1,"coq:exn.The-relation-\u2018ident\u2019-is-not-a-declared-transitive-relation.-Maybe-you-need-to-require-the-Stdlib.Classes.RelationClasses-library","RelationClasses library"]],"This command is just asserting the names of arguments of \u2018qualid\u2019. If this is what you want, add ': assert' to silence the warning. If you want to clear implicit arguments, add ': clear implicits'":[[41,2,1,"coq:warn.This-command-is-just-asserting-the-names-of-arguments-of-\u2018qualid\u2019.-If-this-is-what-you-want,-add-':-assert'-to-silence-the-warning.-If-you-want-to-clear-implicit-arguments,-add-':-clear-implicits'.-If-you-want-to-clear-notation-scopes,-add-':-clear-scopes'"," If you want to clear notation scopes, add ': clear scopes'"]],"This hint is not local but depends on a section variable":[[60,2,1,"coq:warn.This-hint-is-not-local-but-depends-on-a-section-variable.-It-will-disappear-when-the-section-is-closed"," It will disappear when the section is closed"]],"Type of \u2018qualid\u2019 seems incompatible with the type of \u2018qualid\u2019. Expected type is: \u2018type\u2019 instead of \u2018type\u2019":[[71,2,1,"coq:warn.Type-of-\u2018qualid\u2019-seems-incompatible-with-the-type-of-\u2018qualid\u2019.-Expected-type-is:-\u2018type\u2019-instead-of-\u2018type\u2019.-This-might-yield-ill-typed-terms-when-using-the-notation"," This might yield ill typed terms when using the notation"]],"Unable to apply lemma of type "..." on hypothesis of type "..":[[58,0,1,"coq:exn.Unable-to-apply-lemma-of-type-\"...\"-on-hypothesis-of-type-\"...\"","""]],"Unused variable \u2018ident\u2019 might be a misspelled constructor. Use _ or _\u2018ident\u2019 to silence this warning":[[46,2,1,"coq:warn.Unused-variable-\u2018ident\u2019-might-be-a-misspelled-constructor.-Use-_-or-_\u2018ident\u2019-to-silence-this-warning.",""]],"\u2018ident\u2019 already exists":[[28,0,1,"coq:exn.\u2018ident\u2019-already-exists.-(Axiom)"," (Axiom)"],[32,0,1,"coq:exn.\u2018ident\u2019-already-exists.-(Definition)"," (Definition)"],[32,0,1,"coq:exn.\u2018ident\u2019-already-exists.-(Theorem)"," (Theorem)"]],"\u2018qualid\u2019 should go from Byte.byte, (list Byte.byte), or PrimString":[[71,0,1,"coq:exn.\u2018qualid\u2019-should-go-from-Byte.byte,-(list-Byte.byte),-or-PrimString.string-to-\u2018type\u2019-or-(option-\u2018type\u2019)","string to \u2018type\u2019 or (option \u2018type\u2019)"]],"\u2018qualid\u2019 should go from Number.int to \u2018type\u2019 or (option \u2018type\u2019). Instead of Number.int, the types Number.uint or Z or PrimInt63.pos_neg_int63 or PrimFloat.float or Number":[[71,0,1,"coq:exn.\u2018qualid\u2019-should-go-from-Number.int-to-\u2018type\u2019-or-(option-\u2018type\u2019).-Instead-of-Number.int,-the-types-Number.uint-or-Z-or-PrimInt63.pos_neg_int63-or-PrimFloat.float-or-Number.number-could-be-used-(you-may-need-to-require-BinNums-or-Number-or-PrimInt63-or-PrimFloat-first)","number could be used (you may need to require BinNums or Number or PrimInt63 or PrimFloat first)"]],"\u2018qualid\u2019 should go from \u2018type\u2019 to Number.int or (option Number.int). Instead of Number.int, the types Number.uint or Z or PrimInt63.pos_neg_int63 or Number":[[71,0,1,"coq:exn.\u2018qualid\u2019-should-go-from-\u2018type\u2019-to-Number.int-or-(option-Number.int).-Instead-of-Number.int,-the-types-Number.uint-or-Z-or-PrimInt63.pos_neg_int63-or-Number.number-could-be-used-(you-may-need-to-require-BinNums-or-Number-or-PrimInt63-first)","number could be used (you may need to require BinNums or Number or PrimInt63 first)"]],"\u2018qualid\u2019 should go from \u2018type\u2019 to T or (option T), where T is either Byte.byte, (list Byte.byte), or PrimString":[[71,0,1,"coq:exn.\u2018qualid\u2019-should-go-from-\u2018type\u2019-to-T-or-(option-T),-where-T-is-either-Byte.byte,-(list-Byte.byte),-or-PrimString.string","string"]],"\u2018string\u2019 cannot be interpreted as a known notation in \u2018ident\u2019 entry":[[71,0,1,"coq:exn.\u2018string\u2019-cannot-be-interpreted-as-a-known-notation-in-\u2018ident\u2019-entry.-Make-sure-that-symbols-are-surrounded-by-spaces-and-that-holes-are-explicitly-denoted-by-\"_\""," Make sure that symbols are surrounded by spaces and that holes are explicitly denoted by "_""]],"\u2018string\u2019 cannot be interpreted as a known notation":[[71,0,1,"coq:exn.\u2018string\u2019-cannot-be-interpreted-as-a-known-notation.-Make-sure-that-symbols-are-surrounded-by-spaces-and-that-holes-are-explicitly-denoted-by-\"_\""," Make sure that symbols are surrounded by spaces and that holes are explicitly denoted by "_""]],"package-name":[[59,0,1,"coq:exn.package-name.foo-and-not-foo_plugin","foo and not foo_plugin"]],"plugin name anymore":[[59,0,1,"coq:exn.plugin-name-anymore.-Plugins-should-be-loaded-using-their"," Plugins should be loaded using their"]]},objnames:{"0":["coq","exn","Coq exn"],"1":["coq","tacn","Coq tacn"],"2":["coq","warn","Coq warn"],"3":["coq","cmd","Coq cmd"],"4":["coq","flag","Coq flag"],"5":["coq","thm","Coq thm"],"6":["coq","opt","Coq opt"],"7":["coq","attr","Coq attr"],"8":["coq","table","Coq table"],"9":["coq","tacv","Coq tacv"]},objtypes:{"0":"coq:exn","1":"coq:tacn","2":"coq:warn","3":"coq:cmd","4":"coq:flag","5":"coq:thm","6":"coq:opt","7":"coq:attr","8":"coq:table","9":"coq:tacv"},terms:{"0":[2,3,4,5,7,8,9,10,11,12,13,14,25,26,27,28,29,30,31,34,35,36,37,41,43,44,46,50,51,52,53,54,55,57,58,59,60,62,64,66,67,71,72,74,75,77],"00":53,"000":[17,53],"0000000000000002":27,"00075471":77,"00076024":77,"00076039":77,"001":[54,64],"001u":[54,64],"002":64,"002u":64,"00816703":77,"01":[17,53],"013":54,"018":54,"019":53,"02":[17,29,53,77],"02451322":77,"026":53,"027":53,"028":53,"02e":[17,29],"03":[8,17,53],"032":64,"0380":17,"03ff":17,"04":53,"05":17,"0515":77,"052":54,"0530":77,"055":64,"055u":64,"05ef":17,"06":[17,24,53,77],"068":53,"069":53,"07":[17,77],"079":54,"08":[17,77],"09":17,"0beta":25,"0m00":53,"0m03":53,"0m04":53,"0s":71,"0x":29,"0x2a":17,"0xap12":29,"0xb":17,"1":[0,1,2,3,4,5,6,7,8,9,10,11,12,13,14,15,16,18,19,20,21,22,23,25,26,27,28,29,30,31,32,33,34,35,36,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,68,69,70,71,72,73,74,75,76,77],"10":[2,5,24,25,29,31,52,54,57,59,60,64,71,74,77],"100":[17,54,60,64,71],"1000":[62,64],"100000":29,"1000000":29,"1000000000000000000000000000000000":29,"1000000000000000000000000000000001":29,"10002":17,"10008":17,"10012":17,"10014":17,"10017":17,"10019":17,"10022":17,"10049":17,"10053":17,"10059":17,"10061":17,"1007":77,"10076":17,"10085":17,"10088":17,"10095":17,"101":14,"10108":17,"10110":17,"10111":17,"10112":17,"10117":17,"10156":17,"10167":17,"10173":17,"10180":17,"10185":17,"10202":17,"10205":17,"10215":17,"1024":2,"10245":17,"10277":17,"10289":17,"10291":17,"102e":17,"10301":17,"10302":17,"10305":17,"10318":17,"10324":17,"10331":17,"10336":17,"10343":17,"10360":17,"10361":17,"10366":17,"10390":17,"10399":17,"104":77,"10400":17,"10407":17,"10430":17,"10439":17,"10441":17,"10445":17,"10471":17,"10476":17,"10486":17,"10489":17,"10494":17,"105":17,"10577":17,"10592":17,"10614":17,"10651":17,"10657":17,"10664":17,"10728":17,"10731":17,"10739":17,"10747":17,"10750":17,"10757":17,"10758":17,"10760":17,"10762":17,"10765":17,"10772":17,"10774":17,"10796":17,"10803":17,"10806":17,"10811":17,"10812":17,"10816":17,"10824":17,"10827":17,"10832":17,"10842":17,"10852":17,"10858":17,"1088":77,"10891":17,"10894":17,"10895":17,"10897":17,"10899":17,"10904":17,"10912":17,"10932":17,"10947":17,"10956":17,"10963":17,"10965":17,"10966":17,"10970":17,"10971":17,"10985":17,"10988":17,"10996":17,"10997":17,"10998":17,"11":[2,24,25,34,53,57,60],"110":60,"11000":17,"11011":17,"11014":17,"11018":17,"11024":17,"11025":17,"11030":17,"11033":17,"11039":17,"11048":17,"11052":17,"11058":17,"11063":17,"11068":17,"11069":17,"11070":17,"11080":17,"11081":17,"11090":17,"11091":17,"11098":17,"11099":17,"11102":17,"11113":17,"11114":17,"11120":17,"11121":17,"11123":17,"11127":17,"11128":17,"11131":17,"11132":17,"11136":17,"11162":17,"11164":17,"11172":17,"11183":17,"11185":17,"11187":17,"11191":17,"11203":17,"11227":17,"11231":17,"11233":17,"11235":17,"11237":17,"11240":17,"11241":17,"11242":17,"11245":17,"11249":17,"11254":17,"11255":17,"11258":17,"11261":17,"11263":17,"11270":17,"11276":17,"11277":17,"11280":17,"11288":17,"11295":17,"113":17,"11301":17,"11302":17,"11311":17,"11314":17,"11329":17,"11331":17,"11335":17,"11337":17,"11350":17,"11353":17,"11357":17,"11360":17,"11361":17,"11362":17,"11368":17,"11370":17,"11394":17,"11396":17,"11400":17,"11402":17,"11404":17,"11409":17,"11414":17,"11415":17,"11422":17,"11423":17,"11428":17,"11429":17,"11430":17,"11436":17,"11447":17,"1145":77,"11471":17,"11474":17,"11486":17,"11503":17,"11504":17,"11506":17,"11522":17,"11523":17,"11530":17,"11534":17,"11537":17,"11546":17,"11579":17,"1158":77,"11585":17,"11586":17,"11589":17,"11590":17,"11595":17,"11600":17,"11601":17,"11602":17,"11604":17,"11606":17,"11617":17,"11618":17,"11631":17,"11650":17,"11663":17,"11665":17,"11686":17,"11689":17,"117":77,"11705":17,"11718":17,"11720":17,"11725":17,"11727":17,"11740":17,"11741":17,"11742":17,"11746":17,"11755":17,"11760":17,"11761":17,"11766":17,"11783":17,"11795":17,"11797":17,"118":10,"11811":17,"11812":17,"11816":17,"11828":17,"11841":17,"11848":17,"11851":17,"11859":17,"11866":17,"11869":17,"11871":17,"11877":17,"11880":17,"11882":17,"11883":17,"11885":17,"11890":17,"11891":17,"11903":17,"11905":17,"11906":17,"11909":17,"11913":17,"11914":17,"11943":17,"11944":17,"11946":17,"11948":17,"11957":17,"11958":17,"11960":17,"11961":17,"11962":17,"11963":17,"11970":17,"11972":17,"11976":17,"11981":17,"11986":17,"11988":17,"11992":17,"12":[11,25,29,53,54,57,58,60,71],"120":[51,71],"12001":17,"12005":17,"12006":17,"12008":17,"12011":17,"12014":17,"12015":17,"12018":17,"12023":17,"12026":17,"12027":17,"12031":17,"12033":17,"12034":17,"12035":17,"12037":17,"12044":17,"12045":17,"12060":17,"12068":17,"12070":17,"12073":17,"12076":17,"12091":17,"12093":17,"12094":17,"12096":17,"12097":17,"12099":17,"12103":17,"12106":17,"12109":17,"12116":17,"12120":17,"12121":17,"12126":17,"12129":17,"12139":17,"12146":17,"12148":17,"12150":17,"12152":17,"12157":17,"12159":17,"12162":17,"12163":17,"12172":17,"12186":17,"12196":17,"12197":17,"12200":64,"12210":17,"12211":17,"12213":17,"12218":17,"12223":17,"12224":17,"12228":17,"12233":17,"12234":17,"12237":17,"12239":17,"12240":17,"12246":17,"12253":17,"12254":17,"12255":17,"12256":17,"12257":17,"12258":17,"12263":17,"12266":17,"12286":17,"12287":17,"12288":17,"12295":17,"12296":17,"123":71,"12317":17,"12322":17,"12323":17,"12324":17,"12326":17,"12330":17,"12332":17,"12348":17,"12358":17,"12365":17,"12366":17,"12368":17,"12387":17,"12388":17,"12389":17,"12399":17,"12411":17,"12414":17,"12418":17,"12420":17,"12422":17,"12423":[17,54],"12425":17,"12454":17,"12467":17,"12479":17,"12483":17,"12484":17,"12513":17,"12516":17,"12521":17,"12523":17,"12525":17,"12537":17,"12541":17,"12552":17,"12556":17,"12562":17,"12567":17,"12571":17,"12572":17,"12575":17,"12582":17,"12583":17,"12586":17,"12594":17,"12595":17,"126":53,"12613":17,"12647":17,"12648":17,"12653":17,"12677":17,"12678":17,"12682":17,"12683":17,"12685":17,"12707":17,"12708":17,"12716":17,"12738":17,"12752":17,"12754":17,"12755":17,"12756":17,"12762":17,"12765":17,"12768":17,"12770":17,"12772":17,"12773":17,"12775":17,"12777":17,"12787":17,"12793":17,"12794":17,"12799":17,"128":2,"12801":17,"12803":17,"12806":17,"1281":77,"12813":17,"12816":17,"12827":17,"12837":17,"12845":17,"12846":17,"12847":17,"12857":17,"12860":17,"12861":17,"12862":17,"12871":17,"12874":17,"128mb":51,"128u":53,"12908":17,"12946":17,"12948":17,"12950":17,"12960":17,"12965":17,"12972":17,"12975":17,"12979":17,"12984":17,"12986":17,"12992":17,"13":[24,25,51,54,57,77],"13004":17,"13007":17,"13011":17,"13016":17,"13018":17,"13026":17,"13028":17,"13040":17,"13062":17,"13063":17,"13067":17,"13071":17,"13078":17,"13080":17,"13092":17,"13096":17,"13106":17,"13139":17,"13145":17,"13150":17,"13155":17,"13157":17,"13165":17,"13166":17,"13183":17,"13188":17,"13189":17,"13202":17,"13216":17,"13217":17,"13232":17,"13235":17,"13236":17,"13237":17,"13244":17,"13247":17,"13255":17,"13265":17,"13266":17,"13278":17,"13287":17,"13288":17,"13290":17,"13296":17,"13298":17,"13301":17,"13303":17,"13307":17,"13312":17,"13317":17,"13330":17,"13331":17,"13336":17,"13337":17,"13339":17,"13344":17,"13345":17,"13349":17,"13351":17,"13352":17,"13354":17,"13356":17,"13363":17,"13365":17,"13373":17,"13376":17,"13381":17,"13383":17,"13384":17,"13386":17,"13387":17,"13388":17,"13394":17,"13403":17,"13405":17,"13408":17,"13413":17,"13415":17,"13417":17,"13428":17,"13432":17,"13436":17,"13442":17,"13448":17,"13456":17,"13458":17,"13459":17,"13460":17,"13468":17,"13469":17,"1347":17,"13473":17,"13480":17,"13484":17,"13490":17,"13495":17,"135":77,"13501":17,"13509":17,"13512":17,"13517":17,"13519":17,"13541":17,"13550":17,"13556":17,"13559":17,"13562":17,"13563":17,"13566":17,"13568":17,"13579":17,"13581":17,"13582":17,"13586":17,"13589":17,"13617":17,"13618":17,"1362":17,"13624":17,"13654":17,"13671":17,"13696":17,"13699":17,"136u":53,"137":27,"13702":17,"13715":17,"13724":17,"13725":17,"13727":17,"13741":17,"13758":17,"13759":17,"13760":17,"13761":17,"13762":17,"13763":17,"13764":17,"13774":17,"13778":17,"13781":17,"13783":17,"13804":17,"13810":17,"13812":17,"13822":17,"13830":17,"13837":17,"1384":24,"13840":17,"13842":17,"13849":17,"13852":17,"13853":17,"13859":17,"1386":24,"13867":17,"1387":24,"13870":17,"13871":17,"13876":17,"13882":17,"13885":17,"13895":17,"13909":17,"13911":17,"13912":17,"13914":17,"13920":17,"13927":17,"13939":17,"1394":24,"13942":17,"13952":17,"13955":17,"13964":17,"13965":17,"13966":17,"13967":17,"13969":17,"13976":17,"13977":17,"13986":17,"13996":17,"13997":17,"13998":17,"14":[24,25,51,53,57,64],"14005":17,"14006":17,"14007":17,"14008":17,"14009":17,"14011":17,"14012":17,"14015":17,"1402":24,"14023":17,"14024":17,"14033":17,"14037":17,"1404":24,"14041":17,"14059":17,"14070":17,"14081":17,"14083":17,"14086":17,"14087":17,"14089":17,"14090":17,"14092":17,"14093":17,"14094":17,"14096":17,"14100":17,"14102":17,"1412":24,"14124":17,"14125":17,"14128":17,"14137":17,"14138":17,"14141":17,"14148":17,"14153":17,"14174":17,"14183":17,"14189":17,"14207":17,"14208":17,"14211":17,"14234":17,"14238":17,"14256":17,"14257":17,"14258":17,"14260":17,"14261":17,"14263":17,"14265":17,"1427":24,"14283":17,"14285":17,"14289":17,"14293":17,"143":[17,53],"14305":17,"14309":17,"14310":17,"14314":17,"14317":17,"14336":17,"14343":17,"14345":17,"1435":24,"1437":24,"14371":17,"14374":17,"14377":17,"14378":17,"14379":17,"14382":17,"14384":17,"14386":17,"14392":17,"14395":17,"143u":64,"14406":17,"14408":17,"14425":17,"14439":17,"14446":17,"14452":17,"14457":17,"14458":17,"14486":17,"14493":17,"145":[14,53],"14505":17,"14513":17,"14525":17,"14527":17,"14528":17,"14529":17,"14539":17,"14548":17,"14558":17,"14563":17,"14571":17,"14573":17,"14574":17,"1459":24,"14596":17,"146":14,"1460":24,"14601":17,"14606":17,"14609":17,"14610":17,"14644":17,"14650":17,"14651":17,"14652":17,"14657":17,"14660":17,"14662":17,"14664":17,"14666":17,"14668":17,"14669":17,"14670":17,"14671":17,"14672":17,"14673":17,"14678":17,"14679":17,"14683":17,"14685":17,"14687":17,"14693":17,"14695":17,"14696":17,"14697":17,"14699":17,"14705":17,"14708":17,"14713":17,"14718":17,"14722":17,"14731":17,"14732":17,"14734":17,"14736":17,"14750":17,"14758":17,"14780":17,"14787":17,"14801":17,"14802":17,"14809":17,"14813":17,"14819":17,"14841":17,"14843":17,"14844":17,"14848":17,"14863":17,"14872":17,"14874":17,"14879":17,"14892":17,"14899":17,"14901":17,"14907":17,"14928":17,"14930":17,"14938":17,"14940":17,"14957":17,"14959":17,"14963":17,"14967":17,"14975":17,"14984":17,"14986":17,"14989":17,"14996":17,"15":[2,13,25,52,53,57,59,66],"150":[17,55],"15015":17,"15020":17,"15043":17,"15046":17,"15056":17,"15059":17,"15070":17,"15072":17,"15075":17,"15076":17,"15078":17,"15081":17,"15085":17,"15098":17,"15099":17,"151":77,"15121":17,"15122":17,"15139":17,"15171":17,"15193":17,"15194":17,"152":77,"15204":17,"15206":17,"15214":17,"15215":17,"15220":17,"15221":17,"15244":17,"15245":17,"15250":17,"15256":17,"15268":17,"15272":17,"15274":17,"15277":17,"15279":17,"15280":17,"15289":17,"15291":17,"15294":17,"153":53,"15300":17,"15314":17,"15322":17,"15333":17,"15334":17,"15335":17,"15338":17,"15340":17,"15347":17,"15355":17,"15366":17,"15378":17,"15382":17,"15385":17,"15388":17,"15397":17,"15403":17,"15410":17,"15411":17,"15412":17,"15420":17,"15424":17,"15426":17,"15427":17,"15432":17,"15434":17,"15442":17,"15446":17,"15448":17,"15451":17,"15483":17,"15494":17,"15496":17,"15497":17,"15498":17,"155":14,"15511":17,"15526":17,"15527":17,"15531":17,"15532":17,"15537":17,"15554":17,"15559":17,"15560":17,"15567":17,"15568":17,"15575":17,"15577":17,"15578":17,"15581":17,"15596":17,"15597":17,"15599":17,"15600":17,"15606":17,"15612":17,"15619":17,"15620":17,"15621":17,"15628":17,"15633":17,"15634":17,"15637":17,"15644":17,"15650":17,"15652":17,"15653":17,"15657":17,"15662":17,"15668":17,"15669":17,"15675":17,"15683":17,"15690":17,"15693":17,"157":53,"15714":17,"15719":17,"15725":17,"15728":17,"15733":17,"15741":17,"15745":17,"15752":17,"15754":17,"15760":17,"15778":17,"15788":17,"15789":17,"15799":17,"15802":17,"15814":17,"15838":17,"15839":17,"15843":17,"15853":17,"15861":17,"15864":17,"15866":17,"15867":17,"15873":17,"15882":17,"15884":17,"15886":17,"15888":17,"15893":17,"15903":17,"15912":17,"15921":17,"15933":17,"15938":17,"15939":17,"15945":17,"15947":17,"15964":17,"15965":17,"15967":17,"15983":77,"15984":17,"15986":17,"15996":17,"15e":17,"16":[2,25,53,54,57,59,60,71],"160":14,"16004":17,"16005":17,"16007":17,"16015":17,"16023":17,"16026":17,"16030":17,"16040":17,"16046":17,"16062":17,"16063":17,"16066":17,"16069":52,"16070":17,"16096":17,"161":14,"16101":17,"16106":17,"16118":17,"16126":17,"16135":17,"16141":17,"16142":[17,52],"16158":17,"16168":17,"16179":17,"16184":17,"16186":17,"162":[14,53],"16203":17,"16217":17,"16224":17,"16230":17,"16258":17,"16262":17,"16268":17,"16282":17,"16287":17,"16288":17,"16289":17,"16293":17,"163":[53,77],"16302":17,"16308":17,"16322":17,"16323":17,"16329":17,"16340":17,"16355":17,"16375":17,"16395":17,"16407":17,"16409":17,"16411":17,"16413":17,"16414":17,"16415":17,"16418":17,"16429":17,"16434":17,"16436":17,"16438":17,"16440":17,"16466":17,"16472":17,"16479":17,"16485":17,"16489":17,"16498":17,"165":14,"16512":17,"16519":17,"16531":17,"16535":17,"16536":17,"16537":17,"16538":17,"16540":17,"16547":17,"16552":17,"16556":17,"16571":17,"16588":17,"16602":17,"16605":17,"16632":17,"16645":17,"16651":17,"16655":17,"16659":17,"16670":17,"16677":17,"16686":17,"16690":17,"16725":17,"16731":17,"16738":17,"16740":17,"16743":17,"16752":17,"16756":17,"16757":17,"16764":17,"16765":17,"16768":17,"16785":17,"16788":17,"16796":17,"168":14,"16817":17,"16829":17,"16831":17,"16837":17,"16842":17,"16843":17,"16845":17,"16850":17,"16859":17,"16874":17,"16890":17,"16892":17,"169":[14,17],"16902":17,"16903":17,"16904":17,"16906":17,"16909":17,"16910":17,"16911":17,"16914":17,"16915":17,"16918":17,"16920":17,"16925":17,"16926":17,"16929":17,"16931":17,"16937":17,"16945":17,"16947":17,"16957":17,"16958":17,"16959":17,"16960":17,"16981":17,"16988":17,"16989":17,"16991":17,"16992":17,"16994":17,"16996":17,"16997":17,"16999":17,"16th":[24,77],"17":[24,25,27,53,57],"170":14,"17008":17,"17010":17,"17013":17,"17015":17,"17021":17,"17022":17,"17023":17,"17027":17,"17035":17,"17036":17,"17038":17,"17042":17,"17045":17,"17050":17,"17069":17,"17071":17,"17073":17,"17079":17,"17082":17,"17090":17,"17094":17,"17108":17,"17110":17,"17113":17,"17114":17,"17115":17,"17116":17,"17117":17,"17118":17,"17123":17,"17137":17,"17138":17,"17172":17,"17173":17,"17174":17,"17206":17,"17217":17,"17221":17,"17232":17,"17258":17,"17270":17,"17274":17,"17281":17,"17285":17,"17295":17,"173":[2,14],"17303":17,"17304":17,"17305":17,"17316":17,"17318":17,"17321":17,"17322":17,"17324":17,"17333":17,"17344":17,"17347":17,"17352":17,"17359":17,"17364":17,"17371":17,"17382":17,"17392":17,"17394":17,"174":14,"17403":17,"17411":17,"17417":17,"17427":17,"17430":17,"17451":17,"17452":17,"17467":17,"17468":17,"17475":17,"17477":17,"17478":17,"17484":17,"17488":17,"17489":17,"17491":17,"17495":17,"175":[64,77],"17503":17,"17508":17,"17534":17,"17541":17,"17544":17,"17560":17,"17564":17,"17575":17,"17576":17,"17585":17,"17591":17,"17594":17,"17597":17,"17646":17,"17660":77,"17667":17,"17669":17,"17670":17,"17697":17,"177":54,"17702":17,"17704":17,"17716":17,"17718":17,"17721":17,"17732":17,"17733":17,"17734":17,"17743":17,"17744":17,"17745":17,"17747":17,"17754":17,"17760":17,"17772":17,"17774":17,"17777":17,"17782":17,"17787":17,"17788":17,"17789":17,"17794":17,"17795":17,"17796":17,"17801":17,"17805":17,"17808":17,"17817":17,"17832":17,"17836":17,"17841":17,"17844":17,"17845":17,"17854":17,"17856":17,"17857":17,"17860":17,"17861":17,"17871":17,"17872":17,"17887":17,"17889":17,"17891":17,"17892":17,"17894":17,"17897":17,"17902":17,"17927":17,"17934":17,"17935":17,"17936":17,"17946":17,"17959":17,"17963":17,"17964":17,"17984":17,"17985":17,"17986":17,"17987":17,"17988":17,"17991":17,"17993":17,"17998":17,"18":[4,13,25,57,58,59,60,64],"180":54,"18004":17,"18005":17,"18006":17,"18008":17,"18014":17,"18017":17,"18022":17,"18025":17,"18026":17,"1803":17,"18032":17,"18038":17,"18059":17,"18067":17,"18068":17,"18076":17,"18077":17,"18082":17,"18089":17,"18094":17,"18095":17,"18096":17,"18102":17,"18104":17,"18106":17,"18139":17,"18151":17,"18152":17,"18157":17,"18158":17,"18159":17,"18163":17,"18164":17,"18165":17,"18172":17,"18176":17,"18183":17,"18190":17,"18193":17,"18194":17,"18195":17,"18197":17,"18209":17,"18212":17,"18223":17,"18224":17,"18230":17,"18239":17,"18243":17,"18248":17,"18254":17,"18270":17,"18273":17,"18281":17,"18292":17,"18293":17,"18298":17,"18299":17,"18311":17,"18325":17,"18327":17,"18331":17,"18342":17,"18351":17,"18359":17,"18370":17,"18374":17,"18380":17,"18392":17,"18393":17,"18395":17,"184":77,"18411":17,"18424":17,"18432":17,"18434":17,"18442":17,"18444":17,"18445":17,"18447":17,"18448":17,"18449":17,"18458":17,"18463":17,"1850":53,"18500":17,"18501":17,"18503":17,"18507":17,"18516":17,"18523":17,"18524":17,"18527":17,"18536":17,"18537":17,"18538":17,"18539":17,"18544":17,"18548":17,"18550":17,"18551":17,"18556":17,"18558":17,"18560":17,"18563":17,"18564":17,"18565":17,"18576":17,"18577":17,"18580":17,"18588":17,"1859":17,"18590":17,"18591":17,"18594":17,"18596":17,"18599":17,"186":17,"18601":17,"18604":17,"18616":17,"18618":17,"18628":17,"18630":17,"18635":17,"18636":17,"18640":17,"18641":17,"18649":17,"18656":17,"18657":17,"18662":17,"18668":17,"18670":17,"18682":17,"18690":17,"18705":17,"18706":17,"18707":17,"18713":17,"18716":17,"18717":17,"18725":17,"18729":17,"18741":17,"18743":17,"18754":17,"18757":17,"18764":17,"18765":17,"18766":17,"18769":17,"18770":17,"18771":17,"18772":17,"18785":17,"18818":17,"18834":17,"18852":17,"18863":17,"18867":17,"18873":17,"18880":17,"18887":17,"18895":17,"18906":17,"18909":17,"18910":17,"18914":17,"18915":17,"18920":17,"18921":17,"18929":17,"18936":17,"18940":17,"18942":17,"18945":17,"18947":17,"18951":17,"18958":17,"18960":17,"18973":17,"18983":17,"18988":17,"18989":17,"18th":24,"19":[24,25,41,54,57,77],"19006":17,"19016":17,"19017":17,"19027":17,"19032":17,"19040":17,"19049":17,"19060":17,"19069":17,"19082":17,"19088":17,"19092":17,"19096":17,"19099":17,"19100":17,"19115":17,"1912":17,"19129":17,"19136":17,"19137":17,"19138":17,"19141":17,"19144":17,"19149":17,"19152":17,"19153":17,"19164":17,"19166":17,"19179":17,"19188":17,"19197":17,"192":53,"19201":17,"19204":17,"19213":17,"19216":17,"19229":17,"19250":17,"19254":17,"19257":17,"19262":17,"19263":17,"19269":17,"19277":17,"19295":17,"19296":17,"19300":17,"19310":17,"19327":17,"19329":17,"19360":17,"19361":17,"19362":17,"19370":17,"19378":17,"19382":17,"19383":17,"19390":17,"19417":17,"19428":17,"19436":17,"19473":17,"19479":17,"19483":17,"19501":17,"19515":17,"19517":17,"19519":17,"19528":17,"19541":17,"1955":77,"1956":17,"19575":17,"1958":77,"19589":17,"19590":17,"1960":24,"19614":17,"19621":17,"19624":17,"19630":17,"19640":17,"1965":24,"19653":17,"19655":17,"19658":17,"19661":17,"19668":17,"19671":17,"19673":17,"19675":17,"19678":17,"197":77,"1970":24,"19703":17,"19704":17,"1972":77,"19730":17,"19748":17,"19749":17,"19750":17,"19752":17,"19767":17,"19768":17,"19773":17,"1980":77,"1981":77,"1982":77,"1983":24,"1984":24,"1985":[24,77],"1986":[24,77],"1987":24,"1988":[24,77],"1989":[24,77],"1990":[24,77],"1991":[24,77],"1992":[24,77],"1993":[24,77],"1994":[24,77],"1995":[24,77],"1996":24,"1997":77,"1998":[24,77],"1999":24,"19th":24,"1_000_000":29,"1a":54,"1b":54,"1beta":25,"1cvaclvffya5r":51,"1gamma":25,"1p_1":34,"1st":[24,27,34,46,57,59,64,71,72],"2":[0,1,2,3,4,5,6,7,8,9,10,11,12,13,14,15,16,18,19,20,21,22,23,25,26,27,28,29,30,31,32,33,34,35,36,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,68,69,70,71,72,73,74,75,76,77],"20":[2,25,46,57,67,77],"200":[17,52,71],"2000":[17,77],"2001":[24,77],"2002":[24,77],"2003":24,"2004":17,"2005":77,"2006":17,"2007":77,"2008":[17,77],"2010":17,"2011":[17,77],"2013":77,"2015":[17,24],"2016":17,"2017":17,"2018":17,"2019":[17,77],"2020":17,"2021":[17,77],"2022":17,"2023":17,"2024":17,"2034574":77,"2034798":77,"2051":77,"207":77,"208":53,"2080":17,"2089":17,"209":77,"20x":17,"21":54,"2100":17,"2104":17,"212":77,"214f":17,"216":77,"2168":17,"2188":17,"2190":17,"21ff":17,"22":[10,12,54,57,71],"2200":17,"2236":17,"228":77,"22ff":17,"22nd":24,"2300":17,"231":53,"2336":17,"235":77,"2357":17,"236u":53,"237":77,"2372":8,"239":53,"23ff":17,"24":[11,17,44,53,77],"240":51,"246":77,"2489":17,"24th":24,"25":[11,44,64],"2500":17,"252":77,"25379":77,"255":[27,51],"2555":17,"256":2,"256mb":51,"25th":24,"26":[53,54,77],"2600":17,"262":17,"2642":51,"2680":17,"2693":17,"26ff":17,"27":[53,54],"2700":77,"28":77,"2828":17,"285":17,"28756":54,"2884":17,"28x":11,"29":60,"2900":17,"297f":17,"2_5":77,"2a00":17,"2aff":17,"2ap":17,"2nd":[24,34,41,46,57,67,72,77],"2x":[5,11],"2y":5,"3":[0,1,2,3,4,5,6,7,8,9,10,11,12,13,14,15,16,18,19,20,21,22,23,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,72,73,74,75,76,77],"30":[11,17,24,27,71],"300":[17,24],"3051":17,"31":[17,27],"3115":17,"3132":17,"3166":17,"31st":24,"32":[2,17,36,51,53,66],"3209":17,"3219":17,"328":77,"3282":17,"3290316":77,"32mword":51,"33":53,"337720":53,"337876":53,"34":[11,53,71,77],"3415":17,"3434341":77,"345":77,"3479":17,"3488":17,"35":[17,27,53],"3527":17,"3556":17,"356":17,"357":77,"36":57,"3613":17,"362":77,"3632":17,"3659":17,"37":[53,77],"3763":77,"377":77,"3826":17,"384":17,"387":52,"3886":17,"3889":17,"3890":17,"39":[17,53,71],"3941":17,"3943":17,"394648":53,"394700":53,"395448":53,"39634":77,"3977":17,"3989":17,"3994":17,"3em":[26,31,34,35,38],"4":[0,1,2,3,4,5,6,7,8,9,10,11,12,13,14,15,16,18,19,20,21,22,23,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],"40":[14,17,27,41,71],"400":17,"4007":17,"4013":17,"4041":14,"4045":14,"4056":17,"4069":17,"4095":17,"4097":17,"41":[17,51,53,57],"4105":17,"4123":17,"4129":17,"414":17,"4156":17,"4167":17,"421":17,"4250":17,"43":[17,53,54],"4306":17,"4369":17,"4373":17,"4398":17,"44":17,"4413":17,"4415":17,"4416":17,"4436":17,"4450":17,"4476":64,"4495":17,"45":[17,77],"450":17,"4502":77,"4503":17,"4504":17,"4506":17,"4511":17,"45184":53,"4519":17,"4522":17,"4529":17,"4530":17,"4533":17,"4537":17,"4540":17,"4542":17,"4544":17,"4547":17,"4548":17,"4555":17,"4574":17,"4580":17,"4582":17,"4588":17,"4591":17,"4593":17,"4596":17,"46":[11,77],"4603":17,"4606":17,"4607":17,"4608":17,"4614":17,"4623":17,"4627":17,"4630":17,"4632":17,"4638":17,"4644":17,"4673":17,"4677":17,"4683":17,"4690":17,"4696":17,"47":53,"470":17,"4709":17,"4712":17,"4718":17,"4720":17,"4721":17,"4725":17,"4738":17,"4741":17,"4747":17,"4752":17,"4754":17,"4762":17,"4769":17,"4776":64,"4777":17,"4780":17,"48":[17,51],"4818":17,"4822":17,"4823":17,"4824":17,"4832":17,"4841":17,"4844":17,"4851":17,"4858":17,"4863":17,"4871":17,"4876":17,"4880":17,"4881":17,"4882":17,"4887":17,"4890":17,"49":77,"4911":17,"4912":17,"4925":17,"4947":17,"4969":17,"4970":17,"498":66,"4994":17,"4beta":25,"4beta2":25,"4th":[24,41,44,77],"5":[0,1,2,3,4,5,6,7,8,9,10,11,12,13,14,15,16,18,19,20,21,22,23,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],"50":[17,27,41,42,44,53,57,59,71,77],"500":17,"5001":17,"5007":17,"5008":17,"5019":17,"5026":17,"5030":17,"5043":17,"5062":17,"5065":17,"5077":17,"5095":17,"5097":17,"51":17,"5102":17,"512":2,"5123":17,"5127":17,"5132":17,"5150":17,"5155":17,"5159":17,"5163":17,"5173":17,"52":53,"5205":17,"522":17,"5222":17,"5223":17,"5233":17,"52335":77,"5239":17,"5244":17,"5248":17,"5255":17,"5275":17,"5300":17,"5304":17,"5308":17,"5315":17,"5336":17,"5351":17,"5360":17,"5365":17,"5369":17,"5377":17,"5380":17,"5384":17,"5390":17,"5394":17,"54":17,"540":77,"5414":17,"5417":17,"5420":17,"5435":17,"5439":17,"5445":17,"5449":17,"5475":17,"5476":17,"5481":17,"5482":17,"5486":17,"5487":17,"55":[17,54],"5501":17,"5507":17,"5520":17,"5521":17,"5522":17,"5523":17,"5524":17,"5526":17,"5535":17,"5546":17,"5548":17,"5550":17,"5553":17,"5568":17,"5574":17,"5577":17,"5578":17,"5589":17,"5597":17,"5598":17,"5607":17,"5618":17,"5619":17,"5620":17,"5641":17,"5648":17,"5651":17,"5671":17,"56772":53,"56980":53,"57":17,"5702":17,"5706":17,"5726":17,"5730":17,"5752":17,"5764":17,"5777":17,"581478":77,"581501":77,"582153":77,"582176":77,"59":[17,57],"592":53,"5941":17,"5_13":77,"5beta1":25,"5beta2":25,"5beta3":25,"5d4558edf8f5c2c548a3d96c17820169":17,"5pl1":25,"5pl2":25,"5pl3":25,"6":[2,9,25,29,35,53,54,55,57,58,71,74,77],"60":[27,53],"6042":17,"6092":17,"61":[17,53,54],"6109":17,"6134":17,"6261":17,"6278":17,"63":[5,17,29,36,71],"6332":17,"64":[2,36,51,66],"642":77,"6459":17,"650":[17,24,54],"66":[53,77],"664":77,"6677":17,"6705":17,"6714":17,"6720":17,"6785":17,"68":53,"6857":17,"69":[53,71],"6914":17,"6976":17,"6beta1":25,"6f62bda":17,"6th":24,"7":[2,11,25,54,57,64,71,74,75,77],"70":[17,27,36,42,57,71,72],"7015":17,"7017":17,"7086":77,"709":77,"7093":17,"71":46,"7135":17,"72":46,"720":77,"7221":17,"7253":17,"7309":17,"7333":17,"7348":17,"7385":17,"7393":17,"74":53,"7443":17,"7462":17,"75":[17,27,71],"7522":17,"75277":77,"75285":77,"754":[17,36],"757":17,"7615":17,"7632":17,"7634":17,"7674":17,"7675":17,"7695":17,"7697":17,"7698":17,"772":17,"7723":17,"7725":17,"7730":17,"7766":17,"7769":17,"7791":17,"78":59,"7812":17,"7825":17,"7886":17,"7894":17,"7902":17,"7911":17,"7913":17,"7916":17,"7979":17,"7982":17,"7998":77,"7edelahay":77,"7x":11,"8":[2,4,13,24,25,27,30,35,41,51,52,53,54,57,58,59,60,64,66,71,75],"80":[27,71],"8032":17,"8062":17,"8080":17,"8094":17,"8161":17,"8171":17,"8176":77,"82":77,"8215":17,"8217":17,"8252":17,"8276":17,"836":53,"8365":17,"8388607":17,"8388851":17,"84":77,"8402":17,"8419":17,"8451":17,"8457":17,"8459":17,"8481":54,"8488":17,"85":[27,53,71,77],"8540":17,"8555":17,"8560":17,"8638":17,"8642":17,"8649":17,"8667":17,"8669":17,"87":[24,53],"872":17,"8739":17,"874":17,"8764":17,"8779":17,"8791":17,"88":[24,53,77],"8808":17,"8815":17,"8817":17,"8819":17,"8820":17,"8829":17,"8850":17,"8855":17,"8859":75,"8870":17,"8898":17,"89":[53,77],"8905":17,"8920":17,"8945":17,"8965":17,"8987":17,"8989":17,"8991":17,"8_62":77,"8th":24,"9":[2,24,25,29,30,35,53,54,57,64,71,74,77],"9000":17,"9001":17,"9013":17,"9058":17,"9078":17,"9086":17,"9095":17,"9098":17,"91":[7,54,60,77],"9114":17,"9117":17,"9133":17,"9142":17,"9146":66,"9148":17,"9160":17,"9162":17,"92":77,"9214":17,"9270":17,"9274":17,"9279":17,"9288":17,"9294":17,"93":[10,53],"9300":17,"9306":17,"9307":17,"9319":17,"9336":17,"9341":17,"9363":17,"9364":17,"9379":17,"94":77,"9403":17,"9410":17,"9425":17,"947":77,"9490":17,"95":[27,54,60,77],"9508":17,"9509":17,"9512":17,"9514":17,"9517":17,"9519":17,"9521":17,"9524":17,"9530":17,"9532":17,"9555":17,"9569":17,"96":53,"9602":17,"9608":17,"9637":17,"9651":17,"9668":17,"9670":17,"9681":17,"9682":17,"9696":17,"97":[53,77],"9705":17,"9711":17,"9716":17,"9725":17,"9741":17,"9743":17,"9767":17,"9772":17,"978":77,"9803":17,"9811":17,"9816":17,"9825":17,"9829":17,"9840":17,"9844":17,"9848":17,"9851":17,"9854":17,"9856":17,"9867":17,"9872":17,"9874":17,"9876":17,"9883":17,"9884":17,"9885":17,"99":[17,27,71],"9906":17,"9918":17,"9939":17,"996":77,"9964":17,"9971":17,"9979":17,"9984":17,"9995":17,"9996":17,"9_":71,"9_26":77,"9_47":77,"9e":77,"9th":77,"\u00e0":[17,24,55],"\u00e8":77,"\u00e9":77,"\u00e9cole":24,"\u00e9lie":17,"\u00eb":77,"\u015ferb\u0103nu\u0163\u0103":17,"\u03b1":[3,14,25,54,55,57],"\u03b2":[17,25,26,57],"\u03b2\u03b4\u03b9":11,"\u03b2\u03b4\u03b9\u03b6":[0,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],"\u03b2\u03b4\u03b9\u03b6\u03b7":[14,26,31,34,35],"\u03b2\u03b9":[17,41,57,64],"\u03b2\u03b9\u03b6":64,"\u03b2v":55,"\u03b3":[14,26,31,34,35,38,55],"\u03b3_":[26,34],"\u03b3_1":[26,34],"\u03b3_2":26,"\u03b3_c":[26,34,35,38],"\u03b3_i":[26,34,35,38],"\u03b3_n":34,"\u03b3_p":[26,34,35],"\u03b4":[25,26,37,41,57,64,67],"\u03b6":[25,26,57],"\u03b7":[12,17,25,30],"\u03b7\u03b6":57,"\u03b9":[25,26,34,41,55,64],"\u03bb":[17,24,26,31,34,38,52,54,57,66,77],"\u03bbp":34,"\u03bbprolog":63,"\u03bbs":52,"\u03bbx":[26,31,34],"\u03bbz":34,"\u03c0":52,"\u03c1":57,"\u03c3":[35,67],"\u03c6":[17,64,71],"\u03c9":77,"\u2115":39,"a\u2081":4,"a\u2096":4,"abstract":[2,4,5,11,13,14,17,24,25,26,27,28,29,34,35,38,42,44,54,55,58,59,64,67,71],"andr\u00e8":17,"ar\u00eda":17,"arma\u00ebl":17,"bj\u00f6rn":17,"boolean":[2,5,9,11,13,14,17,24,25,27,29,34,37,39,40,42,55,59,60,62,64,67,71],"break":[10,12,17,28,29,30,52,57,59,64,66,71,73,74],"byte":[17,24,25,27,51,59,66,71],"c\u00e9dric":17,"case":[0,1,2,3,4,6,7,8,9,10,11,12,13,14,15,16,17,18,19,20,21,22,23,25,26,27,28,29,30,31,32,33,34,35,36,37,38,39,41,42,43,44,45,46,47,48,49,50,51,53,54,55,56,59,60,61,62,63,64,65,66,68,69,70,71,72,73,74,75,76,77],"cast\u00e9ran":[17,77],"catch":[3,17,25,42,46,57],"char":[2,17,53],"chargu\u00e9raud":17,"chrz\u0105szcz":[17,24],"cl\u00e9ment":[3,17],"class":[13,17,24,25,27,28,35,39,42,44,57,59,60,62,64],"const":[26,34,37,54],"cr\u00e9gut":24,"d\u00e9mon":24,"d\u00e9monstrat":77,"d\u00e9n\u00e8":17,"default":[2,3,4,5,8,9,10,11,12,13,14,17,24,25,27,28,29,32,34,35,37,38,43,44,51,52,53,54,55,57,58,59,60,62,64,66,67,71,74,75],"do":[2,3,4,7,8,10,13,14,17,24,25,27,29,31,32,34,35,37,38,42,46,51,52,53,55,57,58,59,60,62,63,64,66,67,71,74,75],"double":57,"export":[3,5,9,11,13,17,24,27,29,35,38,51,52,54,55,59,60,71],"f\u03c9":24,"f\u2081":4,"f\u2096":4,"f\u2099":4,"filli\u00e2tr":[2,17,24,77],"final":[2,3,4,5,6,8,9,10,11,13,14,17,24,25,27,29,35,40,51,52,53,54,57,59,64,66,67,71,75],"float":[14,17,24,25,34,59,71],"formalis\u00e9":24,"fr\u00e9d\u00e9ric":[5,17,57],"fr\u00e9deric":17,"fran\u00e7oi":[17,57],"franti\u0161ek":17,"function":[2,3,5,9,10,11,12,13,14,17,24,25,26,27,31,33,35,36,37,39,42,45,46,51,52,55,57,58,59,62,64,67,71,73,77],"g\u00e1sp\u00e1r":17,"g\u00e9rard":[24,77],"g\u00f6teborg":24,"ga\u00ebtan":17,"gim\u00e9nez":[24,77],"gr\u00e9goir":[11,17],"gr\u00f6bner":[7,17],"grabovsk\u00fd":17,"gu\u00e9neau":17,"hu\u1ef3nh":17,"ident\u2081":46,"ident\u2099":46,"import":[2,3,4,5,6,7,9,11,13,17,24,25,26,27,28,29,31,32,34,35,36,38,40,42,43,44,51,52,53,54,55,57,58,59,60,62,64,66,67,71,72],"int":[2,3,17,27,36,55,71,75],"j\u00e9r\u00f4me":24,"jes\u00fa":17,"judica\u00ebl":24,"ko\u0161\u00edk":17,"l\u00e9chenet":17,"l\u00e9o":17,"l\u00f6f":[24,27,34],"laulh\u00e8r":24,"leli\u00e8vr":17,"lo\u00efc":[7,17,24],"long":[8,14,17,25,30,51,52,53,58,59,67,71],"march\u00e9":[17,24],"mat\u011bj":17,"math\u00e9matiqu":24,"mu\u00f1oz":[24,77],"new":[4,5,6,8,10,13,14,15,25,27,29,31,32,34,36,37,39,42,43,46,51,52,54,55,58,60,61,64,66,67,71,72,73,75,77],"null":[17,24,27,57],"p\u00e9drot":17,"public":[14,17,25,50,59,74],"q\u2081":17,"q\u2082":17,"r\u00e9alis":24,"r\u00e9gi":17,"rapha\u00ebl":17,"return":[0,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],"s\u00e9bastien":17,"sa\u00efbi":[4,24],"short":[8,14,17,24,25,31,35,36,38,51,53,55,57,59,64,75],"st\u00e9phane":17,"static":[17,24,25,53,71],"sup\u00e9rieur":24,"super":64,"switch":[3,8,13,14,17,24,25,51,53,66],"synth\u00e8s":24,"t\u2081":4,"t\u2098":4,"t\u2099":4,"th\u00e8se":77,"th\u00e9o":17,"th\u00e9ori":77,"th\u00e9ry":[11,17,24],"throw":[17,55],"tr\u1ea7n":17,"triangleright_\u03b2":31,"triangleright_\u03b4":[31,35],"triangleright_\u03b6":31,"triangleright_\u03b7":31,"triangleright_\u03b9":34,"true":[2,4,5,7,9,11,12,13,14,17,24,26,27,34,35,36,37,40,41,44,46,51,53,54,55,57,58,59,62,64,67,71,74],"try":[2,3,11,14,17,24,25,34,35,40,41,43,46,53,55,57,60,62,64,66,67,71],"trzci\u0144ski":17,"u\u2081":4,"u\u2098":4,"universit\u00e9":77,"v\u1d62":55,"v\u2080":55,"v\u2081":4,"v\u2099":[4,55],"var":[17,24,26,54,58],"void":17,"w\u2081":51,"w\u2099":51,"while":[2,3,4,9,10,12,13,14,17,24,25,26,27,28,29,31,32,33,34,35,36,37,40,41,42,43,44,46,51,52,53,54,55,57,58,59,60,62,63,64,66,67,71,73],"x\u1d62":55,"x\u2080":55,"x\u2081":4,"x\u2096":4,"x\u2099":[4,55],A:[3,4,5,7,9,10,11,12,13,17,24,25,26,27,28,29,30,31,32,34,36,37,38,39,40,41,42,43,44,46,50,51,52,53,54,55,57,59,60,62,63,64,66,71,72,74,75,76,77],And:[42,51,53,54,71],As:[2,3,5,6,9,10,11,13,14,17,26,28,30,34,36,37,38,41,42,43,44,46,51,52,53,54,55,57,58,59,60,66,67,71,72],At:[8,11,14,24,26,27,33,34,42,51,52,54,55,57,59,60,71,74],BE:2,Be:[17,75],But:[2,11,17,34,39,41,46,51,53,54,64,75],By:[3,4,5,11,12,13,14,17,29,34,37,44,46,51,53,54,55,57,60,64,66,67,71],For:[2,3,4,5,7,8,9,11,12,13,14,16,17,24,26,27,28,29,30,31,34,35,36,37,38,40,41,42,43,44,45,46,51,52,53,54,55,57,58,59,60,62,64,66,67,71,72,75],IF:[17,71],IS:71,If:[2,3,4,5,7,8,9,10,11,13,14,17,26,28,29,30,32,34,35,37,38,39,41,42,44,46,51,52,53,54,55,57,58,59,60,62,64,66,67,71,72,73,74,75],In:[0,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,56,57,58,59,60,61,62,63,64,65,66,67,68,69,70,71,72,73,74,75,76,77],Is:[25,66],It:[2,3,4,5,6,7,8,9,10,11,12,13,14,17,24,25,27,28,29,30,31,32,34,35,37,38,40,41,42,44,46,51,52,53,54,55,57,58,59,60,62,64,66,67,71,72,74,75],Its:[3,11,17,24,52,55,57,60,67,74],NO:57,No:[3,5,6,9,11,12,13,14,17,24,25,26,30,34,35,36,40,42,44,54,55,57,58,59,60,62,64,66,67,71,72,74],Not:[11,17,27,32,44,51,52,54,55,58,64,67,72,75,77],Of:[2,14,42,51,57],On:[3,10,12,17,24,27,30,32,37,40,44,46,51,52,53,54,57,58,64,71],One:[3,8,9,13,14,17,25,31,32,34,37,38,39,44,51,53,54,55,59,60,64,66,67,71,75],Or:[12,17,41,53,58,71],Such:[12,30,35,42,44,53,55,59,71,75],TO:2,That:[3,27,29,30,34,36,52,54,55,58,64,66],The:[2,3,4,5,6,8,9,10,12,13,14,15,17,24,25,28,29,30,31,32,33,36,37,38,39,40,41,42,43,46,52,54,55,58,59,60,62,63,64,65,66,67,72,73,74,76,77],Their:[3,17,32,34,39,55,57,59,71],Then:[2,4,5,11,14,24,26,27,29,32,34,41,42,46,51,53,54,55,57,58,59,60,64,65,66,67,71,74,75],There:[4,9,10,11,14,17,24,25,26,27,28,29,34,37,38,39,40,44,46,51,52,53,54,55,57,58,59,60,63,64,66,67,71,72,75],These:[3,11,13,14,17,24,25,27,28,29,31,32,34,36,37,38,40,52,53,54,55,57,58,60,64,66,67,71,72,73],To:[3,4,5,6,7,8,9,10,13,14,17,24,25,27,29,30,32,34,37,39,41,42,44,46,51,52,53,54,55,57,58,59,64,66,67,71,72,74,75],WITH:35,With:[3,4,13,14,17,46,53,57,58,67,71],_0:17,_1:35,_:[0,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],__arith:5,__ff:5,__varmap:5,__wit:5,__x1:5,__x2:5,_a_:57,_and_:24,_assoc:59,_b_:57,_complet:72,_coqproject:[17,25,51,52],_correct:72,_darc:51,_e:71,_emphas:75,_eqn:17,_equat:72,_f:[41,72],_foo:17,_full:17,_h:29,_hl:[0,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],_ho:29,_hyp_:57,_i:[35,71],_ind:[34,35,40,71,72],_invol:17,_involut:17,_l:[17,34],_list:71,_list_sep:71,_m:35,_morphism:3,_mybool_scop:41,_n_:57,_not_:17,_p:71,_pack:42,_r:[17,41],_rec:[2,34,35,40,71,72],_rect:[2,17,34,35,40,71,72],_scope:71,_sind:[34,35,40,71],_subproof:[17,59,66],_subterm:59,_tcc:72,_termin:72,_underscores_:17,_x:[46,57],_x_:[17,57],_xxx_:57,a0:[24,46,67],a1:[3,27,34,46,57,58,71],a2:[3,27,34,58],a3:27,a_1:[26,34,35,38],a_:34,a_i:[26,34],a_j:[34,35],a_k:[34,35],a_l:26,a_left:17,a_m:34,a_n:[34,38],a_p:34,a_r:34,a_right:17,aac:17,aaron:17,ab:[17,27,57,67,71],abadi:77,abandon:17,abbr:17,abbrevi:[4,5,13,14,17,24,25,27,32,35,38,59,74],abc:71,abdullah:17,abel:77,abezoutn:57,abhishek:17,abidin:77,abil:[2,3,11,12,13,17,30,52],abl:[3,8,11,13,14,17,24,25,34,42,44,46,51,53,55,57,58,59,61,62,67],abort:[3,11,17,34,42,44,54,55,57,64,66,67],about:[2,3,5,11,13,14,15,17,24,25,29,30,34,37,39,41,51,52,53,54,55,57,58,59,60,62,64,66,67,72],abov:[2,3,5,11,13,14,17,24,28,30,34,37,38,42,44,51,52,53,54,55,57,58,59,64,66,71,72,75],abr:24,abridg:57,abruptli:52,absenc:[9,17,71],absent:[37,59],absolut:[17,24,35,51,53,55,71],absurd:[5,27,34,51,58],absurd_hyp:17,absurd_set:27,abus:[2,55],ac19:[12,77],academ:77,acc:[17,27,34,35],acc_in:34,acc_ind:34,acc_intro:27,acc_inv:27,acc_it:17,acc_iter2:17,acc_rec:34,acc_rect:[17,27,34],acc_simul:17,acc_sind:34,acceler:[17,52],accept:[2,3,13,17,24,28,29,30,32,34,40,44,45,46,51,52,53,54,55,57,58,60,64,66,71,72],access:[2,5,14,17,24,25,27,28,32,33,34,35,36,38,44,51,52,53,55,57,59,71],accessopaqu:17,accident:[17,57],accommod:[24,57],accompani:17,accomplish:[14,57],accord:[2,11,17,26,34,35,41,51,53,55,57,59,60,64,71],accordingli:[8,17,40],account:[5,9,13,14,17,24,26,34,37,41,44,54,57,60,67,71],accumul:54,accur:[17,52,53,57,71],accustom:57,acdsimpl:11,achiev:[7,11,13,17,24,54,57,71],achil:54,ack0:60,ack1:60,ack2:60,ack:[59,60],ackermann:59,ackm:59,acknowledg:25,acm:77,aco:17,across:[17,52,54,55,57,59,73],act:[9,17,37,46,52,54,55,67],actic:77,action:[17,24,52,53,57,60],activ:[8,9,14,17,24,25,29,32,35,37,42,43,44,46,52,53,54,59,60,64,66,71],actual:[2,3,5,8,11,14,17,24,34,37,42,43,44,46,54,55,57,60,64,67,71,72],acycl:[24,39],aczel:24,ad:[2,4,9,13,14,17,24,25,27,29,34,37,42,44,51,53,54,55,57,58,59,60,62,64,66,67,71,73,75,77],adam:17,adapt:[3,7,17,24,51,57,63],add1:[55,64],add:[3,4,5,8,9,10,11,13,14,17,24,25,27,29,31,32,34,37,41,42,44,46,51,53,54,55,57,58,59,60,62,64,66,67,71,73,75],add_0_l:17,add_assoc:[17,59],add_bottom:[17,71],add_carri:17,add_carry_div2:59,add_comm:[3,17,59,64],add_instance_attempt:42,add_last:57,add_mul:57,add_shuffle0:59,add_shuffle1:59,add_shuffle2:59,add_shuffle3:59,add_succ_comm:59,add_top:[17,71],add_transpose_neqkei:17,add_un_double_moins_un_xo:17,add_zifi:5,addit:[3,4,5,8,9,13,17,24,25,27,29,31,34,35,39,51,52,53,54,55,58,59,62,64,65,66,67,71,72,73],addition:[9,13,14,17,34,46,53,54,58,59,64,66],addn0:57,addn:57,addnc:57,addnca:57,addpath:[17,24],addr:17,addrecpath:[17,24],address:[17,52],addsn:57,addsnn:57,addx:57,adhoc:[17,37],adjac:57,adjoin:17,adjoint:17,adjointif:17,adjust:[14,17,38,71],admiss:[30,38],admit:[8,9,13,17,30,32,37,42,46,51,52,57,66],admitaxiom:17,adopt:[17,57,73,75],adrian:17,advanc:[5,17,25,33,34,42,53,54,58,64,71,74],advantag:[8,17,24,46,51,53,57,62,64,67],advertis:17,advic:[15,17],advis:[11,17,24,25,28,29,30,54,60],aeq:3,aesthet:54,affect:[12,17,24,29,34,41,44,46,53,54,55,57,59,60,64,66,71],affeldt:17,aforement:[9,51],aft:75,after:[2,4,5,7,9,11,13,17,24,29,32,34,35,38,41,42,46,51,52,53,54,55,57,58,59,60,62,64,66,67,71,72],afterward:[9,17,41,44,52,57,60,66,67],again:[3,13,17,24,34,42,52,53,55,57,60,64,66,71],against:[10,13,17,44,54,57,58,59,60,62],agda:30,aggress:57,ago:17,ahead:[17,54],aid:24,aim:66,aka:[17,72],akin:[17,30,55],akira:17,al:[3,57],al_unit:54,ala:53,alban:17,albeit:17,aleksandar:77,alessandro:77,alexand:17,alexandr:17,alexei:17,algebra:[7,14,17,24,39,42,54,55,64,77],algorithm:[3,7,9,11,13,17,24,25,41,51,54,57,59,62,66,77],algorithmica:77,ali:17,alia:[2,17,24,29,35,46,55,58,60],alias1:35,alias2:35,alias:[2,17,24,25,29,35,55],alias_definit:[55,58],align:[10,59,71],all:[2,3,4,5,7,8,9,10,11,12,13,14,17,24,26,27,28,29,30,31,34,35,36,37,38,39,40,41,42,44,46,51,52,53,54,55,57,58,59,60,62,64,66,67,71,72,73],all_eq:12,all_iff_morph:3,all_nul:57,all_sig2_cond:17,allai:17,alldfil:53,allevi:67,alloc:[17,51],allow:[2,3,4,5,7,8,9,10,11,12,13,14,17,24,25,26,27,28,29,30,31,32,34,37,38,40,42,44,46,51,52,53,54,55,57,58,59,60,62,63,64,66,67,71,72],allt:[17,24],alltact:52,almost:[3,17,57,67,75],alon:[17,24,34,67],along:[8,17,24,34,53,57,58,66,74],alongsid:17,alpha:[17,31,54,55],alpha_p:5,alphabet:[17,60],alreadi:[2,4,13,17,24,27,28,32,37,41,42,44,51,52,53,54,55,57,58,59,60,66,67,71,73],alright:2,also:[2,3,4,5,6,7,8,9,10,11,12,13,14,17,24,25,26,27,28,29,30,31,32,34,35,37,38,39,40,41,42,43,44,46,51,52,53,54,55,57,58,59,60,62,63,64,66,67,71,72,73,74,75,77],alt:[17,52],alter:[17,35,75],altern:[7,8,9,11,13,17,24,25,29,30,35,40,43,44,46,52,53,55,57,59,62,64,65,66,71,75,77],although:[3,5,9,17,35,37,53,55,57,58,60,64,66],alvarado:24,alwai:[2,3,4,6,9,10,11,12,13,14,17,24,26,34,35,37,41,42,44,51,52,53,54,55,57,58,60,66,67,71,74,75],am:55,ambient:55,ambigu:[4,17,25,46,53,57,59,60,66,71],ambiti:24,ambrois:17,amen:67,amend:42,amin:17,aminev:17,amokran:[4,24],among:[7,13,17,24,25,26,34,44,53,54,55,57,64],amorim:17,amount:[3,5,8,14,17,27,51,54,58],an:[2,3,4,5,6,7,8,9,10,11,12,13,14,17,24,25,26,27,28,29,30,31,32,34,36,37,38,39,40,41,42,43,44,46,51,52,53,54,55,58,60,62,63,64,66,71,72,74,75,77],ana:17,analog:[3,17,34,54,57,58,66],analogu:57,analys:13,analysi:[17,24,25,30,34,37,40,46,57,58,72,77],analyz:[17,27,40,57,67],anand:17,ancestor:[24,53],andE:57,and_assoc:59,and_darc:51,and_rect2:27,andb:[2,13,17,27,62],andb_comm:59,andb_negb_l:17,andb_prop:59,andb_true_intro:59,andbc:57,andp:57,andpp:17,andr:17,andrea:[17,77],andrej:17,andrew:[17,77],anew:57,angl:24,anguag:77,ani:[2,3,4,5,6,7,8,9,10,11,12,13,14,17,24,26,28,29,30,31,32,34,35,37,38,39,41,42,43,44,46,51,52,53,54,55,57,58,59,60,62,64,66,67,71,75],annoi:57,annot:[3,9,14,17,24,25,27,34,41,42,45,51,53,55,57,66],anomali:[10,17,24,59],anonym:[14,17,24,25,44,54,66],anoth:[3,4,9,11,13,14,17,24,27,31,32,34,35,40,42,43,44,46,51,52,53,54,55,57,58,59,62,63,64,66,67,71],anr:17,ansi:51,answer:[11,46,53],antialias:52,antinomi:24,antipoli:[17,24],antiquot:[17,25],antisymmetr:17,anton:17,antonia:72,antonio:17,anymor:[9,17,55,59],anyth:[2,13,17,35,44,46,51,55,57,58,64,75],anything_ind:2,anything_rec:2,anything_rect:2,anything_sind:2,anytim:54,anywai:57,anywher:[43,58,75],ap:[4,11],apart:[9,13,31,35,55],api:[8,17,25,59,63],app:[17,26,27,34,35,55,58,67],app_ass:17,app_assoc_revers:17,app_eq_app:17,app_eq_con:17,app_inj_pivot:17,app_inj_tail_iff:17,app_inv_head_iff:17,app_inv_tail_iff:17,app_length:17,app_nil_end:17,app_nth2_plu:17,app_rlist:17,appar:[14,17,51,54,57],apparatu:9,appart:51,appcontext:17,appdata:52,appeal:27,appear:[2,6,9,10,11,13,14,17,24,28,29,31,34,35,37,38,39,41,43,44,46,51,52,53,54,55,57,58,59,60,64,66,67,71,74,75],appel:17,append:[3,17,29,35,43,53,54,66,75],append_const:17,append_inj:17,appendix:17,appli:[2,3,4,5,9,10,11,13,14,17,24,25,26,27,28,29,30,31,32,34,35,36,37,38,40,41,42,44,46,51,53,54,55,59,60,62,66,71,72,75],applic:[3,5,10,11,13,14,17,24,25,26,29,30,35,36,37,41,46,52,55,57,59,60,64,66,67,71,72,77],apply_id:71,apply_mor:3,approach:[24,27,52,53,55,57,58,67,75],appropri:[4,13,14,17,29,53,55,57,59,62,64,66,67,75],approxim:[5,12,14,17,60],apr:17,april:[17,77],ar:[2,3,4,5,6,7,8,9,10,11,12,13,14,16,17,24,25,26,27,28,29,30,31,32,33,34,35,36,37,38,39,40,41,42,43,44,46,50,51,52,53,54,55,58,59,60,61,62,63,64,65,67,71,72,73,74,75],ar_unit:54,arab:29,arakaki:17,arbitrari:[2,3,5,10,11,14,17,24,31,44,46,53,57,60,62,71],arbitrarili:[17,58,71],archclean:53,architect:24,architectur:[17,24,29],archiv:[17,77],area:17,aren:[17,52,53,54,58,73,75],arg:[17,24,28,37,44,51,53,55,57,60,67],arg_spec:41,args_modifi:41,argument:[3,4,5,6,7,9,11,12,13,14,17,24,25,27,28,29,30,31,32,33,34,35,38,40,42,43,45,51,52,54,55,58,59,60,62,64,66,72,75],argument_spec:41,ari:[3,17,34],aria:17,aris:[3,9,13,17,30,67,71],arith:[3,5,9,11,17,24,27,43,53,57,58,59,60,64,72],arith_bas:[17,59],arith_prebas:17,arithmet:[17,24,25,36,44,57,60,61,71],arithr:11,ariti:[2,17,24,25,46,55],arnaud:17,around:[12,17,24,29,46,52,53,55,57,58,59,64,67,71,75],arr:[26,34],arrai:[0,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,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],array_get:36,array_set:36,array_typ:36,arrow:[3,4,14,17,52,57,60,64,67],art:[17,52],arthur:17,articl:24,articul:71,artifact:17,artifici:[17,24,67,71],as_ipat:58,as_nam:58,ascand:24,ascii:[17,52,53,71,75],ascii_as_ot:17,asciisyntax:17,ascrib:17,asf:77,asid:[34,64,66,67],asin:17,ask:[2,3,17,25,42,43,53],askra:59,aspect:[17,24,46],asr:17,ass:54,ass_app:17,assert:[2,17,24,25,26,28,34,41,54,55,57,58,62,64,66,67,71],assert_fail:[17,25],assert_succe:[17,25],assia:[11,17,42,57,77],assign:[13,17,25,27,29,43,51,52,53,54,55,58,66,71],assist:[17,24,25,33,65,75],assoc:54,associ:[2,3,11,13,14,17,24,25,26,27,28,29,31,32,34,35,36,37,38,42,44,46,51,52,53,54,55,57,58,59,60,64,66,67],assum:[2,3,5,11,13,17,26,27,28,32,34,35,36,38,39,42,44,46,51,53,54,55,57,58,59,64,66,71,75],assumpt:[4,10,17,24,25,26,32,33,34,35,36,44,51,52,53,54,58,59,60,66,67,77],assumption_token:[28,59],assur:[17,53],ast:[17,24,37],ast_closure_term:17,asterisk:75,asymc:52,asymmetr:[17,46],asymptot:[2,59],async:[8,17,52,54],asynchron:[17,25,66,76],atan_right_inv:17,atom:[4,5,8,14,17,26,60,62,67,71],atomic_tac2pat:55,attach:[14,17,29,52,59,71,74],attack:51,attempt:[8,14,17,24,41,52,54,66],attent:66,attila:17,attr:[17,29,51],attr_valu:29,attract:17,attribtu:14,attribut:[3,5,9,13,14,16,25,28,30,32,34,37,40,41,42,44,51,54,55,59,60,62,64,66,71,74],auger:17,august:[17,24],austin:24,author:[2,3,4,5,7,8,9,11,14,17,27,29,42,46,57,73,74],auto:[11,13,14,17,24,29,34,41,44,51,52,54,57,58,59,60,62,66,67,72],auto_us:60,autoappli:[13,17],autocomplet:17,autogener:17,autoinlin:[2,17],autom:[17,24,25,43,54,59,61,64,66,67,77],automat:[2,3,5,7,9,10,13,14,17,24,25,27,28,35,37,40,42,46,52,53,54,55,57,58,60,64,65,66,71,72,75,77],automath:24,automatiqu:77,automaton:[24,75],autonom:17,autorewit:17,autorewrit:[3,17,24,60],autounfold:[17,60],auxiliari:[8,17,34,53,54,57,66],avail:[2,9,11,12,13,17,24,25,27,30,35,36,37,38,40,42,46,50,51,52,53,54,55,57,58,59,60,62,63,64,65,66,71,72,74,75,76,77],avec:24,averag:24,avi:17,avl:[17,27],avoid:[6,8,11,12,13,17,24,25,29,34,37,52,54,55,57,58,59,60,64,66,67,71,74],awai:[17,54],await:52,awar:[17,51,52,55,58,59,62,66],awk:17,awkward:[24,54],ax:[26,44,67],axiom:[3,7,9,10,11,12,14,17,24,25,27,28,29,30,31,32,34,35,36,38,42,44,51,52,54,57,58,59,60,64,66,67,71,72,74],axiomat:[17,24,27,36,54,71],axiomatis:17,ayach:17,azevedo:17,b0:46,b1:[57,59],b2:[57,59],b2n:[41,59],b2n_le_1:17,b3:57,b:[2,3,4,8,9,10,11,12,13,14,17,24,25,27,28,31,34,35,37,38,40,41,42,44,46,50,51,52,53,54,55,57,59,60,62,64,66,67,71,72,77],b_1:34,b_:34,b_i:34,b_j:34,b_m:34,b_r:34,ba:17,back:[3,9,14,17,24,51,52,54,57,58,59,66,67],backchain:57,backend:24,background:[17,31,51,52,54,66],backport:17,backquot:17,backslash:51,backspac:52,backto:[17,59],backtrac:[17,25,55,59],backtrack:[11,13,17,24,25,52,58,60,67],backward:[17,25,51,52,55,57,63,66,71],bad:[2,11,12,14,17,34,59,64],baeld:17,bahmann:17,bail:8,bakel:17,balaa:72,balanc:[17,57],banner:24,bar0:55,bar81:[26,66,77],bar:[2,8,14,17,29,35,51,52,53,55,57,64,66,71,74],bare:[17,71],barenblat:17,barendregt:[24,77],barra:[11,17,24],barrett:17,barri:17,bart:17,barth:72,base0:60,base1:60,base:[3,5,10,11,12,13,14,17,24,25,29,33,35,39,42,43,44,51,52,53,54,55,57,58,60,62,63,64,66,67,71,73,74,75,77],base_includ:59,basenam:53,bash:[17,52],basi:[7,17,52,59],basic:[3,11,17,24,25,32,33,34,35,37,40,42,44,46,51,58,59,60,63,66,67,73],basicelim:[17,67],basicmatch:46,batch:[8,17,25,54,66],bati:17,battl:2,baz:[14,53],bazaux:53,bdd:2,bdenesgregoire11:[64,77],bear:10,beautifi:[17,51],becam:[17,24],becaus:[2,3,4,8,11,12,14,17,24,26,28,29,31,33,34,35,37,39,40,41,43,44,45,46,51,52,53,54,55,57,58,59,60,62,64,66,67,71,72],beck:17,becker:17,becom:[2,8,11,17,24,26,28,34,35,40,44,46,52,53,55,57,58,59,64,66,67,71],bedrock:17,been:[2,3,8,9,10,11,13,14,17,24,25,27,28,29,32,34,35,41,42,44,46,51,52,53,54,55,57,58,59,60,63,64,66,67,71,72,73,74],beep:71,befor:[2,4,5,13,14,17,28,29,32,34,37,41,42,44,51,52,53,54,55,57,58,59,60,64,66,67,71,73,74,75],beforehand:[17,51,55],begin:[0,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],beginn:[17,25],behalf:17,behav:[3,11,17,24,28,29,31,34,35,43,53,54,55,57,58,60,62,64,67,71],behavior:[2,3,4,11,13,14,17,24,29,30,32,34,41,43,44,51,52,53,54,55,57,58,59,60,64,66,67,71,73,75],behaviour:[2,17,34,38,53],behind:[4,17,28,34,57],being:[2,3,9,11,12,13,14,17,24,32,33,34,35,37,38,40,42,46,51,52,53,54,55,57,59,60,64,66,67,71,72,75],believ:[17,54,55],bell:17,belong:[5,8,11,26,27,29,34,37,39,53,54,57,59,60,63,67,71,75],below:[2,4,5,8,9,10,11,13,14,17,25,26,27,31,34,35,38,40,41,43,51,52,53,54,55,57,59,64,66,71,72,74,75],benaissa:77,benchmark:[17,54],benefici:8,benefit:[13,17,51,57],bengtson:17,benjamin:[11,17,77],benni:17,berlin:77,bernhard:17,bernstein:24,bertholon:17,bertot:[17,24,72],bertrand:17,besid:[3,17,24,34,57],besson:[5,17],best:[13,17,53,54,57,60,71],best_effort:[13,17],beta1:25,beta2:25,beta3:25,beta:[2,11,17,24,55,57,58,64,71,77],betaiota:17,better:[11,14,17,24,51,52,53,57,59,60,64,67,71,72],between:[3,4,10,11,13,14,17,24,25,26,27,29,33,34,38,39,43,44,46,51,52,53,54,57,58,60,64,65,67,71,72,75],bewar:[17,53,55,63,67],beyond:[59,63],bezem:77,bezout_comm:17,bf:[13,17],bfb0037116:77,bfb0040259:77,bformula:5,bg:66,bhat:17,bi:3,bibliographi:25,bibtex:17,bidirect:17,bidirection:[17,25],big:[11,14,17,57,59,71],big_int:17,big_int_z:17,big_prop:57,bigbodi:57,bigger:34,biggest:53,bigint:[17,29,71],bign:17,bignat:[29,71],bignum:[17,53],bigop:57,bigq:17,bigvee_:5,bigwedge_:5,bigwedge_i:5,bigz:[17,53],bij:4,biject:[4,17],bin:[17,53],binari:[3,5,7,11,14,17,24,27,29,37,42,51,53,57,58,60,64,71],binary64:[17,27,36],binary_induct:17,bind:[3,9,10,14,17,24,25,28,32,34,35,37,40,43,44,46,51,54,57,64,66,67,72],binder:[12,13,17,24,25,30,32,34,37,38,40,52,54,55,58,59,63,64,67,75],binder_interp:71,bindir:[17,51],binint:[17,53],binintdef:17,binnat:[17,59],binnatdef:[17,59],binnum:[17,59,71],binop:5,binopspec:[5,17],binpo:[17,59],binposdef:[17,59],binrel:5,bird:6,birkhaus:77,bishop:24,bit0_eqb:59,bit:[2,5,17,27,29,30,34,36,51,53,66,71,75,77],bitvector:17,bitwis:[17,59],blaauwbroek:17,black:[17,29],blacklist:[2,17,59],blah:55,blank:[17,24,29,53],blanqui:57,blaudeau:17,blazi:77,bleed:17,bliss:55,blob:[52,71],block:[2,9,10,14,17,25,29,30,34,37,38,44,46,54,64,65,67],blocktyp:8,blow:17,blowup:17,blue:[29,52],bm:57,bmod:57,bodi:[2,4,6,13,14,17,24,32,35,37,38,41,42,44,51,55,57,58,59,64,72,75],bodin:17,bodo:17,boespflug:77,bogu:8,bohannon:17,bold:66,boldfac:29,boldo:24,book:[17,25],bookkeep:25,bool:[2,4,5,12,13,17,24,27,30,35,36,37,40,41,42,44,46,55,57,58,59,60,71],bool_as_dt:17,bool_as_ot:17,bool_cas:40,bool_choic:[27,59],bool_in_nat:4,bool_ind:[27,40],bool_nat:17,bool_rec:[27,40],bool_rect:[27,40],bool_scop:[17,27,41,71],bool_sind:[27,40],boolean_if_scop:57,boolnot:17,boolord:17,boot:17,border:71,borg:17,boro:17,borrow:17,both:[2,3,4,11,14,17,24,25,26,27,28,29,31,34,37,38,40,42,43,44,46,51,52,53,54,57,58,60,61,64,66,67,73,74],bottom:[3,17,37,46,52,54,55,58,64,71],bottomup:3,bou97:[11,77],boulier:17,bound:[3,5,6,7,10,14,17,24,25,26,27,28,31,32,34,39,41,42,44,46,52,54,55,57,58,59,60,62,64,72],boundari:[17,54],bourk:17,boutilli:17,boutin:[11,24,77],box:[12,17,29,54,71],box_ind:12,box_irrelev:12,box_rec:12,box_rect:12,box_sind:12,boyer:[17,24],brace:[25,44,52,59,71],bracket:[17,24,26,44,54,57,59,66,71,75],braibant:17,brain:17,branch:[2,5,9,17,25,34,40,45,46,55,59,60,66,67,72],brand:17,brandenburg:17,breadth:13,breakag:17,breakpoint:[17,25],breitner:17,bresenham:24,breviti:[42,58,66],bridg:[17,57],briefli:[24,27,57],bring:[17,59],broke:17,broken:[11,17,71],brought:17,brows:[17,25,27,52,57,73],browser:[17,52],bruijn:[17,24,31,33,77],bruno:[11,17,24],brute:[57,64],bs:46,btauto:[17,62],btauto_plugin:[11,27,29,36,57,66],btauto_term:62,buchberg:[7,24,77],buffer:[17,25,35,53],bug:[12,17,24,52,54,66],bugfix:17,buggi:[17,25,33],bugtrack:17,build:[2,5,9,11,14,17,24,25,26,27,32,33,34,37,42,46,51,54,55,57,59,60,63,65,66,67,72,75,76,77],build_:37,build_monad:14,build_monoid:14,build_setoid:42,buildlist:46,built:[2,4,11,17,24,25,26,31,32,34,37,41,42,52,53,54,58,60,61,62,67,71,72],builtin:52,bullet:[8,17,25,34,59,67],bump:17,bunch:[17,57],bundl:17,burden:[3,63],busi:17,button:[8,17,24,52],buys:17,bv2n:17,bvand:17,bvector:17,bveq:17,bvneg:17,bvor:17,bvxor:17,byextend:17,bypass:59,bypass_check:[30,32,34,59],bypass_guard:17,byte_scop:71,bytecod:[12,17,59,64],bytevector:17,c0:[11,59],c1:[17,46,57,67,71],c2:[17,46,57,67,71],c3:[57,71],c4:57,c:[0,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],c_1:[5,26,34,35],c_2:5,c_:34,c_i:[5,34,35],c_k:[26,34],c_m:35,c_n:[34,35],c_pattern:57,c_q:34,cach:[5,12,17],cachan:[17,24],caci:17,caglayan:17,calcul:[24,25,77],calculi:[54,62,77],calculu:[11,14,17,24,25,27,29,31,33,34,35,37,46,54,57,58,62,64,66,67,71,77],call:[2,3,4,5,6,9,11,12,13,14,17,24,25,26,27,28,29,30,31,32,34,35,36,37,39,40,42,44,45,46,51,53,54,57,58,59,60,64,66,67,71,72],callabl:2,callback:[2,17],calvin:17,cambridg:[24,77],came:17,caml:[17,24,75],camlc:53,camldir:17,camlflag:[17,53],camloptc:53,camlp4:[17,24],camlp5:[17,71],camlpkg:[17,53],can:[2,3,4,5,6,7,8,9,10,11,12,13,14,17,24,25,26,27,28,29,30,31,32,33,34,35,36,37,38,39,40,41,42,44,45,46,51,52,53,54,55,57,58,59,60,61,62,63,64,65,66,67,71,72,73,74,75],can_in_comp:17,can_in_pcan:17,cancel:[11,38,41,57,66],candid:[57,58,64,72],cannot:[2,3,4,8,9,10,11,12,13,14,17,26,28,29,32,34,35,36,37,40,41,44,46,51,53,54,55,57,58,59,60,62,64,66,67,71,72,75],canon:[2,4,5,11,13,17,24,25,30,32,34,35,37,38,44,45,53,57,59,71,77],cantor:[17,34],capabl:[3,17,51,53,54,55,64],capit:[17,29,74],captur:[3,17,34,44,57,64,71],car:3,carbonneaux:17,card:57,card_nat:54,cardinal_add_in:17,care:[2,13,14,17,46,53,54,64,67,71,75],carefulli:60,carl:17,carlo:[24,77],carri:17,carrier:[3,11,14,42,57],carst:17,cartesian:[14,54],carthi:60,cascad:17,case_eq:17,case_item:40,case_l_r:17,case_l_r_l:17,case_l_r_r:17,casetyp:17,cast:[2,12,17,25,40,46,54,55,57,58,60,64,71],casual:[25,57],cat:[17,27,74],categor:24,categori:[4,8,13,17,35,51,59,61,74,75],catherin:9,cauchi:[17,27],caught:[46,54,55],caus:[8,12,14,17,32,51,52,53,54,55,57,58,59,63,64,66,71,75],caution:66,caveat:[2,17,25,55,57,60],cbn:[10,17,41,64],cbv:[10,14,17,24,31,57,64],cc:[53,77],cd:[2,17,53],ce:42,ceil:5,cell:36,centaur:24,central:[24,25],centuri:24,cep:17,cequival:3,certain:[4,17,24,29,44,46,51,54,57,58,59,64,67,71],certif:17,certifi:[2,9,17,24,77],cezari:17,cf07:[36,77],cf:[2,9,17,24,29,34,40,42,46,59,67],cfc58:[26,77],ch85:[24,77],ch86a:[24,77],ch86b:[24,77],chailloux:24,chain:[2,17,25,51,64,71,74],chaje:[17,58],challeng:[17,24,77],chalmer:[24,77],chanc:[17,53],chang:[2,4,5,8,9,11,13,14,25,26,28,29,31,34,36,37,38,41,43,51,52,53,54,57,58,59,60,62,63,64,66,67,71,73,74,75],change_arg:17,change_no_check:[17,58,64],changelog:[17,24],changement:24,channel:[17,51],chantal:17,chap:24,chapoton:17,chapter:[2,3,8,9,11,13,15,17,24,26,27,29,31,32,33,34,38,40,42,45,52,54,55,57,58,59,61,63,65,71,73,75,76],char63:[27,36],char_scop:71,charact:[2,8,10,14,17,24,25,27,29,35,36,40,44,46,53,54,55,57,58,59,64,66,71,72,74,75],character:[8,17,34,40,42],characterist:5,charg:17,charset:[52,75],chasl:24,chat:17,chatzikonstantin:17,cheap:17,cheapli:46,check:[2,3,4,5,6,8,9,10,11,12,13,14,17,24,25,26,27,30,32,33,34,35,37,38,39,40,41,42,43,44,46,51,52,53,55,57,58,59,60,62,64,66,67,71,72,74,75],check_guard:59,check_posit:59,check_univers:59,checkabl:24,checkbox:52,checker:[2,9,11,17,24,25,26,29,33,73],checkproof:17,checksum:[17,51],chet:24,chetan:24,chile:17,chines:[2,24],chiron:17,chlipala:17,chluebi:17,cho:17,choic:[3,17,27,34,51,52,55,62,71,75],choice2:27,choicefact:17,choos:[2,3,17,32,34,42,43,52,53,54,57,58,67,71,72,75],chose:53,chosen:[11,34,54,55,57,58,66,71],christian:17,christin:[17,24,27,34,77],christoph:[2,17,24,77],chronolog:15,chung:17,church:[24,77],ci:[11,17,53,57,73],cic:[0,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],circ:27,circular:[4,17,57],circumv:17,cjk:[17,29],clamp:57,claret:17,clarif:17,clarifi:[17,24],clariti:[58,66],clash:[2,17,53,54,57],class_1:17,class_2:17,class_of:42,classic:[11,17,24,25,27,34,51,55,57,66],classical_left:[17,58],classical_prop:17,classical_right:[17,58],classicaldedekindr:17,classicalfact:17,classifi:[17,27],classnam:13,claud:17,claudel:17,claudio:[3,17,24],claus:[9,13,14,17,24,25,28,29,30,32,34,35,40,41,51,53,54,55,57,59,60,62,64,67,71,72],clean:[17,53,57,67,72],cleanal:[17,53],cleaner:17,cleanup:17,clear:[17,24,25,29,38,41,44,54,55,58,64,67,71],clear_switch:57,clearbodi:[17,24,38,58],clearer:55,clearli:[11,24,71,74],clenv_refine_in:17,clerc:17,clever:[17,59,64],click:[8,17,52],client:17,clipboard:52,clock:64,clos_refl_tran:17,clos_t_clos_rt:17,close:[2,3,4,5,7,9,11,14,17,24,28,29,32,34,35,38,44,51,52,55,57,59,60,64,66,67,71,75],closedn:17,closer:[17,24,31,57,60,72],closest:[27,53],closur:[17,24,31,54,55,62,66],club:17,cm:53,cma:17,cmafil:53,cmd:[3,17,38,51,52,54],cmi:17,cmifil:53,cmo:[51,59],cmofil:53,cmorphism:[3,17],cmp:42,cmu:24,cmx:[2,3,5,6,9,11,17,27,29,34,36,42,43,51,54,55,57,58,59,60,64,66,72],cmxa:17,cmxafil:53,cmxfile:53,cmxsfile:53,cn:17,cnet:24,cnr:24,co:[4,10,11,17,24,25,42,44,54,57,59,64,67,71,77],co_high:14,co_low:14,coarser:17,coc:24,coc_histori:17,cockx:77,code:[9,10,11,12,17,24,25,29,33,36,51,52,53,54,55,57,59,60,63,64,71,72,73,74,75],codebas:17,codifi:[55,77],codomain:[17,42,71],coeffici:[7,11,17],coen:[3,17,24],coerc:[4,41,57,60,64],coercibl:[9,57],coercion:[9,13,17,24,25,28,35,37,38,41,42,45,57,58,59,77],coercion_class:[4,71],coexist:17,coffe:17,cofix:[17,25,28,29,31,44,54,55,57,64,67],cofix_bodi:30,cofix_definit:[30,38],cofixpoint:[17,29,30,32,34,38,57,59,64,66],cohen:17,coher:[17,41],coin:5,coinduct:[14,17,25,26,27,32,33,34,37,40,46,59,67,71],collabor:77,collaps:[14,17,51],colleagu:24,collect:[10,17,27,51,53,60,66,72],collid:24,collis:[17,24,51],colog:77,colon:[17,51,53,57,66],color:[8,17,25,51,52,66,75],colson:24,column:[17,46,53,57],com:[2,5,17,51,52,54,71],comand:17,combin:[2,3,5,9,12,14,17,24,25,26,27,29,34,37,40,42,46,52,53,54,55,57,59,63,64,75],combinator:17,combinatori:77,combine_length:17,come:[2,6,8,13,17,24,27,34,43,51,52,54,55,57,59,60,64,71],comextradep:59,comfort:[17,46],comit:17,comma:[17,46,51,52,55,57,74],command:[2,4,5,6,7,8,9,10,11,12,14,16,25,26,27,28,29,30,32,34,36,37,38,40,41,42,43,44,45,46,53,54,55,58,60,62,63,64,72,73,74],commemor:[24,77],comment:[2,5,17,24,25,29,52,54,57,60,66,75],commit:[17,53,54,55],common:[11,14,17,25,26,27,29,31,32,34,42,55,57,60,67,71,74],commonli:[9,14,17,27,40,53,54,55,57,58,66],commun:[2,17,24,27,29,51],commut:[7,11,17,24,44,59],comp:[17,53],compa:17,compact:[17,24,25,34,54,57,59,66,71],compani:[17,66],companion:43,compar:[4,5,11,14,17,24,25,27,37,42,53,54,55,57,58,64,66,67,73],compare_cas:17,compare_cont:17,compare_dec:[17,24],compare_structur:54,comparison:[5,14,17,24,27,42],compat:[2,3,4,13,14,24,25,29,34,42,51,52,53,58,59,62,63,64,71],compatibl:17,compcert:25,compil:[2,3,8,9,10,11,12,24,25,26,27,29,32,35,36,38,46,55,58,64,73,74,75,77],complement:[17,57],complementari:[2,17,24,27,42,57],complet:[3,4,5,6,7,8,9,10,11,17,24,29,30,32,34,36,40,42,51,52,53,54,57,58,59,60,62,66,67,71],completeness_weak:17,complex:[2,11,17,24,25,29,33,35,52,54,55,57,59,61,63,66,67],compli:36,compliant:17,complic:[34,43,46,55],compon:[13,17,24,25,30,33,34,35,37,42,51,52,53,54,57,59,60,71],compos:[3,4,34,44,57,67,71],composit:[3,27,71],compound:[29,54],comprehens:24,compress:[51,53],compris:[3,24],compspec:17,comput:[2,3,7,9,11,17,24,25,27,29,30,32,34,35,36,37,41,42,46,51,52,55,57,59,67,71,72,77],computation:66,con:[0,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],conc:67,concat:[17,46,55],concat_length:17,concat_nil_foral:17,concaten:[17,26,27,54,55,67],concept:[17,24,25,31,57,77],conceptu:[3,34],concern:[2,12,17,24,26],conchon:77,concis:[55,57],concl:[17,59],concl_occ:58,conclud:[5,13,17,34,54,57,64,67],conclus:[3,11,13,17,24,28,34,54,55,57,58,60,64,66,67,71],concret:[2,13,14,17,25,26,29,34,42,46,51,57,64,71],concurr:17,condit:[3,4,9,11,17,24,25,27,30,50,53,59,60,63,64,66,67],cone:[5,17],conejero:17,conf:[17,53],confer:[24,77],confid:[17,24,25],config:[17,51,52],configur:[8,17,24,25,29,40,51,52,59,64,66,73],confin:8,confirm:[59,71],conflict:[17,24,25,46,54,55,71],conflit:17,confluenc:[25,31],conform:17,confus:[4,10,13,17,24,26,29,34,44,46,52,55,57,71],confusingli:[17,58],cong_iff_0:17,cong_iff_ex:17,congr:57,congruenc:[3,12,17,24,25,34,54,62,64,67],congruenceclosur:24,conj:[27,57,58,66,71],conjectur:[17,28,66],conjunct:[3,5,11,17,24,27,34,57,59,60,67,71],conli:27,connect:[17,25,57,62,71],connor:17,conor:[67,77],cons2:34,cons3:34,cons:17,cons_inj_bool:44,cons_inj_nat:44,cons_rlist:17,cons_seq:17,consequ:[17,24,26,29,34,38,39,42,43,44,46,52,57,60],conserv:[2,17],consf:[0,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],consid:[2,3,4,5,9,11,12,13,14,17,24,26,28,29,30,31,34,37,41,42,44,46,52,53,54,55,57,58,59,60,64,67,71,73,75],consider:[3,9,17,37,39,46,64,67,71],consist:[3,4,5,11,13,14,17,24,27,30,31,34,35,52,55,57,58,59,64,65,66,71],consn:46,consol:54,consolid:17,consortium:17,constabl:24,constant:[2,4,5,6,9,10,11,13,14,17,24,25,26,27,30,31,32,34,35,36,38,41,42,44,46,51,54,55,57,58,60,64,66,67,74],constantli:57,constitut:[25,39,55],constr:[3,5,14,17,24,34,42,54,55,57,71],constr_eq:17,constr_eq_nouniv:17,constr_eq_strict:[17,54],constr_may_ev:17,constr_with_bind:17,constrain:[9,14,24,60,67],constraint:[3,5,8,9,10,13,17,24,25,34,35,39,43,44,51,53,54,55,58,67,71],constrast:37,constrexpr:17,construct:[3,4,5,8,9,10,11,13,14,17,25,27,28,29,30,31,33,35,41,42,43,46,52,53,55,57,58,62,63,64,65,66,67,71,77],constructivecauchyr:17,constructiveepsilon:17,constructiveminmax:17,constructivepow:17,constructiver:17,constructor:[2,4,9,10,12,13,14,17,24,25,26,27,30,31,32,35,36,37,40,41,42,43,44,46,54,55,57,58,59,60,62,64,66,71,74],consult:64,consumpt:[8,17,54,55],consw:34,contact:[17,52],contain:[2,5,7,8,10,13,14,15,17,24,27,29,30,31,34,35,38,39,41,42,43,44,46,51,52,53,54,55,57,58,59,60,62,64,66,67,71,72,73,74,75],contains0:67,contains0_ind:67,contains0_sind:67,contant:31,content:[2,17,24,27,32,35,42,51,52,53,54,57,59,66,71,75],context:[4,5,9,10,11,14,17,24,25,26,29,30,31,32,34,35,38,41,43,44,51,52,59,60,62,64,66,67,71],contextu:[17,24,25,31,41],contigu:[17,29],continu:[2,17,24,52,53,54,55,57,71,73],continut:17,contract:[10,17,24,31,34,54,62,71,77],contradict:[17,34,54,57,60,67],contradictori:[17,67],contrainst:17,contrari:[3,4,9,13,17,30,40,44,57,67],contrast:[14,17,34,53,57,60,62,64,67],contrastingli:29,contravari:14,contravariantli:3,contrib:[2,17,24,53,55],contribut:[17,25,53,71],contributor:17,control:[2,3,13,14,16,17,24,25,34,37,41,51,52,53,55,60,62,67,71,75],control_command:[17,29,59],contructor:67,conv:26,conv_expr:17,conveni:[2,4,6,12,17,24,28,29,33,34,35,44,46,52,53,54,57,66,67,71],convent:[2,17,25,33,42,51,57,59,71],convention:[17,53,71],converg:17,convers:[2,3,7,8,9,11,12,13,17,24,25,26,30,32,33,34,35,37,54,55,57,58,60,66,71,75],convert:[3,4,12,13,14,17,25,26,27,34,37,41,44,54,55,57,58,64,67],convert_concl_no_check:17,convinc:24,cook:17,coolen:17,coordin:[17,24],copattern:30,cope:17,copi:[2,17,36,46,52,53,54,57,59,75],coq84:17,coq85:[17,31,77],coq86:[39,77],coq88:17,coq89:[24,77],coq92:[34,77],coq:[2,9,11,13,15,17,25,26,29,30,46,51,53,54,55,57,58,59,63,66,71,72,73,75,76,77],coq_:2,coq_color:[17,51,66],coq_flag:53,coq_makefil:[17,24,25,51,52,59],coq_micromega:5,coq_profile_compon:51,coq_src_subdir:53,coq_vers:53,coqbin:[17,51,53],coqbot:17,coqc:[17,24,25,29,52,54,59,66,75],coqchk:[17,25,53,64,73],coqchkextraflag:53,coqchkflag:[17,53],coqcorelib:53,coqdebug:53,coqdep:[17,25,51,59],coqdev:17,coqdir:[17,75],coqdoc:[17,24,25,51,53,76],coqdocdir:17,coqdocextraflag:53,coqdocflag:[17,53],coqdocid:75,coqdocinstal:[17,53],coqdockw:75,coqdocmodul:75,coqextraflag:53,coqflag:[17,53],coqid:[8,25,35,51,53,54,66,76],coqiderc:[17,52],coqidetop:17,coqlib:[17,51,53,71],coqlib_path:17,coqlib_url:[17,75],coqlibinstal:[17,53],coqmakefil:[17,25,52],coqmakefile_vers:53,coqn:[17,51,53],coqoon:17,coqpath:[17,51,53],coqplugininstal:[17,53],coqpp:[17,53],coqprefixinstal:17,coqprim:17,coqproject:53,coqrc:[24,25],coqremotebrows:17,coqrunbyteflag:17,coqtail:[51,53,66],coqtest_skipcomplex:17,coqtimelog2html:[17,53],coqtoolsbyteflag:17,coqtop:[17,24,25,26,35,52,53,54,59,66],coqtop_toplevel:53,coquand:[24,34,77],coqworkmgr:17,coram:75,corbineau:[17,24],core:[3,13,17,24,25,27,29,41,45,51,53,54,57,59,60,62,65,71],core_scop:[14,71],corecurs:[25,33,71],corn:[24,46,67,77],cornel:24,corner:[17,64],corollari:[17,32],corpu:57,correct:[2,8,9,11,17,24,25,27,28,32,35,46,51,53,57,59,64,66,67,71],correctli:[17,24,29,34,51,52,53,54],correspond:[2,3,8,9,11,13,14,15,17,24,26,27,28,33,34,35,37,38,42,44,46,51,52,53,54,55,57,58,59,60,64,66,67,71,72,75],corrupt:[17,24],cos3pi4:17,coscoi:24,cosin:17,cosmo:77,cost:[17,51,55,60],could:[2,3,4,5,6,11,12,17,24,29,31,34,37,42,46,51,52,55,57,58,60,62,66,71,72,73],couldn:13,count:[13,17,25,51,57,58,59,64,66,67],count_occ:17,count_occ_app:17,count_occ_bound:17,count_occ_elt_eq:17,count_occ_elt_neq:17,count_occ_repeat_eq:17,count_occ_repeat_excl:17,count_occ_repeat_neq:17,count_occ_rev:17,count_occ_sgt:17,count_occ_uniqu:17,countabl:17,counter:[17,62],counterpart:[2,3,9,11,17,27,30,34,57],counterproduct:17,coupl:[11,17,46,53,57,75],courant:24,cours:[2,14,17,24,42,51,52,57,64,71],courtesi:17,courtieu:[17,24],cousineau:24,couterbal:17,covari:14,covariant_ind:14,covariant_rec:14,covariant_rect:14,covariant_sind:14,covariantli:3,cover:[17,44,54,57,65],cp90:[24,34,77],cp:53,cp_phi:11,cpattern:[54,55],cpermut:17,cpow:11,cpp:77,cpu:[17,59],cr_of_q:17,craft:[54,57],craig:77,cran:17,crash:17,crashcoqid:52,creal:17,creat:[3,8,9,13,17,24,25,29,34,38,40,42,51,52,53,54,57,58,59,64,66,67,72,75],creation:[17,24,43,60],credit:[17,24],crelat:3,crelationclass:17,cring:17,cristal:24,cristina:[24,46,67,77],criteria:[2,17,72],criterion:[10,17,33,34,60],critic:[17,24,33,54,59],croap:24,crone:17,cross:[17,24,35,38,64,66,71],cryptograph:24,crzero:17,cs:[17,24],csdp:5,css:[52,75],cst1:17,cst2:17,cst:17,cstop:5,ct95:[67,77],ctan:75,ctcoq:24,ctl:24,ctltctl:24,ctrl:[17,52],ctw21:[10,77],ctx:67,ctx_ind:67,ctx_rec:67,ctx_rect:67,ctx_sind:67,cube:77,culmin:24,cumbersom:[44,55],cumul:[12,13,17,24,25,26,29,30,31,34,37,40,71],cumul_univ_decl:[14,34],cup:[17,26,34,51],cur:54,curiou:5,curli:[8,25,44,59,71],current:[2,3,4,5,8,9,10,12,14,17,24,27,28,29,32,34,35,36,37,38,41,42,44,46,51,52,53,54,55,57,58,59,60,64,66,67,71,75],curri:[17,24,26,66,77],cursor:[17,52,66],custom:[2,3,11,13,17,24,25,27,29,36,53,54,57,59],customiz:17,cut:[14,17,24,25,29,52,57,58,60],cutoff:54,cutrewrit:17,cv:[17,51],cv_infty_cv_0:17,cvc3:17,cvcl:17,cycl:17,cyclic31:17,cyclic:[17,27,64],cyclicaxiom:17,cyprien:17,cyril:[17,29],czajka:17,d0:[67,71],d1:71,d2:71,d:[2,4,5,11,14,17,24,26,34,46,51,52,53,54,57,58,62,67,75,77],d_1:11,d_2:11,d_item:57,d_tactic:57,dabrowski:17,dai:[24,51],daili:55,dalrympl:17,dama:77,dan:[17,24,77],danger:17,daniel:[17,24],danilkin:17,dapprich:17,dark:52,darryl:17,dash:75,data:[17,24,27,34,36,39,53,54,55,57,64,66,77],databas:[3,13,17,25,54,57,62,64],datadir:17,datatyp:[2,17,24,25,26,35,44,46,54,55,57,59,60,67,71],date:[17,24,53],davi:24,david:[17,24,72,77],db72:[26,77],db:[3,17],dc95:[54,77],ddoubl:57,de:[17,24,31,33,59,77],dea:[24,77],deactiv:[9,17,24,25,27,46,59],dead:[24,64],deal:[3,5,8,13,17,24,25,42,46,57,60,64,71,72],debian:17,debug:[2,5,9,13,14,17,24,25,28,52,53,57,58,60,62,64,66,72],debug_univ_nam:14,debugg:[17,24,25],dec:[9,24,46],dec_int_scop:[17,71],dec_uint_scop:[17,71],decad:17,decemb:[17,24,77],decentr:17,decid:[5,8,11,17,24,25,27,29,34,51,53,55,57,60,71],decidableclass:17,decidabletyp:17,decim:[5,17,27,29,59,71],decimalfact:17,decimaln:17,decimalnat:17,decimalpo:17,decimalstr:17,decimalz:17,decis:[2,17,24,25,58,62,64,77],decl_not:[30,34,40,71],declar:[2,4,5,6,7,8,9,10,11,12,14,17,24,25,26,27,28,29,30,31,32,34,35,36,37,43,46,51,53,54,58,59,60,64,71,72,75],declareunicodecharact:75,decnat:29,decod:17,decompos:[24,57,67],decomposit:57,deconstruct:46,decor:[24,29,42],decoupl:[8,17],decreas:[3,7,9,17,30,34,55,59,72],decrement:[17,54],dedekind:17,dedic:[11,17,24,29,36,55,57],deduc:[5,17,44,51,57,58,67],deduct:[5,24,57],deem:[2,51],deep:[17,24,57,67],deep_tupl:46,deepen:13,deeper:[34,46],def:[26,35,67],def_bodi:[4,32,38,42],def_n:57,default_bindings_src:52,default_go:53,default_with:17,defaultrel:3,defect:[25,55],defend:24,defens:[17,24,44,57],defer:[52,55,57],defin:[2,3,4,5,6,7,9,11,12,13,14,17,24,25,26,27,28,29,30,31,32,33,36,38,39,40,41,42,43,44,46,51,52,53,57,58,59,62,64,66,67,71,72,74,77],defined:3,definin:35,definit:[2,4,8,10,11,13,17,24,25,26,27,28,29,31,33,35,36,38,41,42,43,44,51,53,58,59,60,62,66,67,72,73,74,75,77],definition:[4,12,17,31,32,35,37,64],definitionalclass:17,degener:[40,57],degrad:54,degre:[5,73],del00:[54,77],delahay:[24,77],delai:[14,17,25,40,64],deleg:[8,17,25,29],delet:[17,52,54,57,66],delete_on_error:17,deliber:[31,55],delic:34,delimit:[8,17,33,35,41,44,59,66,71,75],deliv:17,delpath:[17,24],delphin:77,delta:[11,17,24,32,35,37,55,64],delta_reduct:[55,64],demand:57,demonstr:[24,54,67],dempski:17,denomin:[11,17,37,71],denot:[3,4,11,17,24,26,28,29,30,34,35,39,40,42,43,52,54,57,58,67,71],denum:11,dep:51,dep_ret_typ:46,depart:3,departur:55,depend:[2,3,7,8,9,12,13,14,24,25,26,27,28,29,30,32,34,35,36,37,38,40,42,43,44,51,52,54,55,57,60,62,64,66,71,72,77],deplaix:17,deploi:17,deprec:[2,4,13,17,25,28,29,32,35,41,51,55,58,59,60,64,66,71,72],depth:[3,5,13,17,29,54,57,58,59,60,62,64,71,75],der:17,derek:77,deriv:[3,5,9,13,17,24,25,26,27,30,34,38,40,54,64,66,73],derive_plugin:6,desarzen:17,describ:[2,3,4,6,7,8,10,11,12,13,14,17,24,27,29,31,32,34,35,36,37,39,40,42,43,46,51,52,53,54,55,57,58,59,64,65,66,67,71,72,75],descript:[17,24,25,27,29,31,38,40,42,46,51,53,57,66,67],design:[2,8,11,17,24,25,37,44,57,64,71,77],desir:[9,11,17,34,52,53,54,57,59,73,75],desktop:17,desmettr:[17,24],despit:[36,57],dest:[4,17],destauto:[17,67],destdir:[17,53],destko:17,destroi:55,destruct:[2,13,17,24,25,34,54,55,57,58,64,71],destruct_bool_and_rewrit:54,destruct_with_eqn:71,destructor:[17,25,30,31,37],destructur:[17,24,25,32,40],destructuring_let:[32,46],desugar:37,detach:[17,52],detail:[3,5,7,14,25,27,31,36,37,41,42,51,52,55,57,58,59,64,66,71,72,74,75],detect:[5,8,17,25,41,44,52,53,57,66],determin:[4,13,17,31,34,36,40,41,43,53,54,57,58,64,66,67,71,72,75],determinist:17,dev:[17,24,51,53,71],develop:[2,3,12,13,14,17,24,25,27,32,35,42,44,51,52,53,54,57,58,59,60,64,66,67,71,74,77],devis:17,devot:[52,57],df:[13,17,60],dfrac:5,di:[54,77],diagnos:14,diagnost:71,diagon:34,diagram:11,dialect:17,dialog:[17,52,65],dialogu:55,did:[8,11,17,26,29,57,58,59,66,67],didn:[3,17,51,53],diff2:77,diff:[17,24,25,51,53,54],diff_failur:17,differ:[3,4,9,11,13,14,15,17,24,25,26,27,29,31,34,35,37,38,41,43,46,51,52,53,54,55,57,58,59,60,62,64,67,71,72,73,75,77],difficult:[11,17,29,55,71,72],difficulti:53,digit:[17,24,27,29,44,51,52,71],dimens:17,dintuit:[17,62,71],dir:[17,51,53,75],direct:[2,9,12,16,17,24,31,34,42,46,52,53,57,58,59,71],directli:[2,3,4,9,13,14,17,24,27,28,34,43,51,52,53,55,57,58,59,60,64,67,72,75],directori:[2,14,17,24,27,35,51,52,53,59,60,71,75],dirpath:[17,35,51,59],disabl:[2,8,9,12,13,14,17,25,28,32,34,35,37,44,51,52,54,57,58,59,64,66],disallow:[12,14,17,37,51],disambigu:[17,44,57,71],disappear:[2,17,24,34,55,60,67,71],discard:[14,17,52,54,55,58,64,75],discharg:[3,14,17,24,25,28,38,72],disciplin:[17,24,26],discontinu:17,discourag:[17,29,32,35,53,54,55,58,59,60,66],discours:[17,52],discov:[17,53],discoveri:24,discrep:[17,57],discret:5,discrimin:[13,17,24,54,57,58,59,60,62,64,66],discrimine:[10,12,46],discrr:[24,27],discuss:[3,17,24,25,54],disembodi:42,disequ:[9,60],disj:[17,71],disjoint:[27,67],disjointed:67,disjunct:[17,25,34,57,58,59,60,67,71],disk:[51,52,53,66],dismiss:67,dispatch:55,displai:[2,9,12,14,16,17,25,35,37,41,42,46,51,53,54,55,57,58,60,64,66],dispos:57,disregard:42,distanc:24,distinct:[9,13,17,26,34,42,44,46,53,54,55,57,60,64,67,71],distinguish:[14,17,24,26,34,37,57,64,71],distr:2,distribut:[11,17,24,25,50,73,75],disus:17,div0:[17,59],div2:[9,17,72],div2_0:17,div2_1:17,div2_decr:17,div2_equ:72,div2_even:17,div2_ind:72,div2_l:72,div2_le_lower_bound:17,div2_le_mono:17,div2_le_upper_bound:17,div2_obligation_1:9,div2_obligation_2:9,div2_obligation_3:9,div2_obligation_6:9,div2_odd:17,div3:9,div:[2,3,5,11,17,27,59],div_exact:59,div_mod:17,div_mod_to_equ:[5,17],div_theori:11,div_zdiv:17,diveq_iff:17,diveucl:2,divex:2,divid:[5,15,17,24,58],divide_gcd_iff:17,divide_to_equ:5,divis:[3,11,17,24,25,57],divisor:[7,17],dj:57,dm82:[55,77],dmitri:17,do_depind:67,do_makefil:24,doc:[17,24,51,53,63,71,74,77],doc_grammar:17,docdir:[17,53],docgram:71,docker:17,docroot:[17,53],doctor:24,doctorat:77,document:[3,8,9,11,12,16,17,24,25,27,42,51,52,54,55,57,59,64,65,66,67,71,72,74,76],doczkal:17,doe:[2,3,4,5,8,9,12,13,14,17,24,25,26,27,29,30,34,35,36,38,39,41,42,44,51,52,53,54,55,57,58,59,60,62,64,66,67,71,72,75],doesn:[4,14,17,27,29,31,35,46,51,52,53,54,55,57,58,59,62,66,67,71,73],doi:77,doligez:24,dom:71,domain:[3,5,11,14,17,24,25,26,34,42,61,64,71],domin:75,dominiqu:17,don:[4,10,13,14,17,28,34,35,37,46,52,53,54,57,58,60,62,64,66],donati:17,done:[2,3,5,6,7,9,10,11,13,17,24,27,29,30,32,34,35,36,38,40,42,43,46,52,53,54,55,57,58,59,60,64,66,67,71,72,75],dont:[17,59],dorel:17,dot:[11,14,17,24,35,37,52,59,71],doubl:[17,24,27,29,34,44,52,53,54,57,59,71,75],double_var:17,doublen:57,dowek:24,down:[3,14,24,25,45,51,52,54,55,57,59],download:[17,27,53,77],dozen:64,dp:[2,17],drag:[17,24],dramat:64,draw:24,drawback:[9,17,67,71],dreyer:77,drive:64,driven:[24,60],driver:5,drop:[3,17,51,54,59,71],drope:17,dstroot:17,dt:60,dtauto:[17,62],dual:[3,9,24,55],dualli:[3,44,57],duboi:17,dudenhefn:17,due:[2,3,13,14,17,24,27,30,34,46,52,54,55,59,64,66,67,71,72,73],dummi:[2,14,17,24,55,77],dummy_ind:14,dummy_rec:14,dummy_rect:14,dummy_sind:14,dump:[5,17,24,51,75],dumpbox:17,dumpgraph:17,dune:[17,25,51,59],dup:[17,57],duplic:[3,11,17,43,57,67,71],duprat:24,durat:51,dure:[2,9,11,13,14,17,24,37,42,46,51,53,54,55,57,58,60,64,66,67,71,72],duti:55,dvdn1:57,dvdn_mull:57,dvdn_mulr:57,dvdn_subr:57,dvdn_tran:57,dvi:75,dx:77,dyc92:[54,62,77],dyckhoff:[24,54,62,77],dynam:[2,11,13,17,25,36,51,59,71],dynlink:[17,59],e0:[42,46,72],e1:[17,42,46,57],e2:[17,42,46],e:[0,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,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],e_1:[5,35],e_2:[5,35],e_:[17,35],e_i:35,e_n:35,e_type_of:17,ea:13,each:[2,3,5,6,8,9,10,11,13,14,17,24,26,27,29,30,34,35,36,37,38,39,40,42,43,44,46,51,52,53,54,55,57,58,59,60,64,66,67,71,72,74,75],eager:17,eagerli:55,eappli:[17,54,58,60,66,67,71],earli:[2,15,17,25,26,54,64],earlier:[8,17,53,54],eas:[13,17,37,53,55,57,58,66],easi:[7,11,13,17,27,46,52,53,60,67],easier:[2,10,17,24,45,52,57,58,67,71],easiest:53,easili:[13,17,53,57,72],eassert:[17,43,58],eassumpt:[17,43,58,60],eauto:[17,25,43,54,57,60],eb:13,ecas:[17,43,58,67],echo:53,econom:[24,77],econstructor:[17,43,67],ecosystem:[25,73,77],ed:[17,24],edestruct:[17,43,58,67],edg:[17,52],edinburgh:24,ediscrimin:[17,43,67],edit:[17,24,25,29,51,53,57,66,71],editor:[17,52,53,77],eduardo:24,edward:17,eelco:77,eeli:17,eelim:[17,43,67],eenough:[17,43,58],eexact:[17,43,58],eexist:[17,43,60,66,67],effect:[2,9,11,13,14,17,24,25,29,30,34,35,38,43,51,52,53,54,57,59,64,66,71,75],effici:[2,11,12,13,17,25,29,36,57,60,64,77],effort:[13,17,24,63,74],eg:[17,53],ei:57,eight:34,einduct:[17,43,58,67],einject:[17,43,67],eintro:[43,58],either:[2,5,8,11,14,17,26,28,29,31,34,35,36,37,39,40,41,44,46,51,52,53,54,55,57,58,59,60,64,66,67,71,74,75],ej:57,el:77,elabor:[13,14,17,25,27,33,37,41,44,45,51,55,58],elaps:54,elast:24,elect:[25,50],electron:[24,77],eleft:[17,43,67],eleg:[2,55,59],elegantli:58,element:[2,3,11,12,17,25,26,27,34,35,36,46,57,59,60,71],elementari:[25,27,57,58,71],elements1:71,elements2:71,elid:57,elim:[5,17,24,25,54,58,67],elim_let:17,elimin:[10,12,14,17,24,25,26,27,30,31,34,35,37,40,54,55,58,67,71,72,77],elimtyp:17,elpi:[17,63],elrod:17,els:[2,4,9,11,12,13,17,29,30,35,40,41,46,52,54,55,57,62,67,71,75],elsevi:77,elsewher:[9,17,52,59,71],elt:5,elt_eq_unit:17,emac:[17,51,52,59,66],email:52,emb:[17,24,71],embed:[24,25,29,71],emerg:24,emilio:17,emit:[2,10,12,13,17,34,53,71,74],emmanuel:24,emp:60,emphas:46,emphasi:25,emploi:[17,42],empti:[2,3,5,7,12,13,17,24,26,34,40,43,51,53,55,57,58,59,60,67,71,72],empty_context:17,empty_neutr:3,empty_set:[17,40,62,71],emptyf:[0,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],emul:[2,12,17,40,57],en:[24,57,64,77],enabl:[2,4,7,8,9,10,11,12,13,14,17,25,34,37,42,51,52,53,54,57,58,59,60,67,75],enable_notation_flag:71,encapsul:57,enclos:[2,29,41,53,54,55,66,71,75],encod:[3,13,17,24,25,27,34,53,71,75],encount:[2,11,17,52,53,54,64],encourag:[17,46,53,54],end:[0,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,35,36,37,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],enforc:[9,12,14,17,26,32,34,44,55,57,58,66,71],engin:[13,17,24,33,43,55,57,58,64,77],english:17,enhanc:[2,17,52,57],enjoi:[31,34,37,57],enough:[10,11,14,17,34,44,57,58,67,71],enrich:[5,17,24,26,27,67],enrico:[8,17,42,57,77],ensur:[2,10,13,14,17,24,27,30,34,39,52,55,59,64,71,72],ensuremath:75,enter:[8,17,25,30,32,34,35,38,44,46,52,54,55,59,60,71],entier:17,entir:[10,13,17,24,25,31,33,34,41,44,52,53,57,60,64,66,71],entri:[17,24,25,28,29,37,51,52,53,54,55,67],enumer:[5,17,34,40],enviro:[17,59],environ:[3,9,11,12,13,14,17,24,25,26,28,30,31,32,34,35,38,42,43,52,53,55,57,60,62,64,66,67,71,72,75],envr:5,ep:60,epos:[17,43,58,71],epsilon:[17,60],epsilon_smallest:17,eq0:3,eq0_le0:44,eq:[3,5,11,14,17,27,35,40,42,54,57,58,59,64,67,71],eq_:27,eq_add_:27,eq_adda_b:57,eq_adda_c:57,eq_big:[17,57],eq_big_:57,eq_bigr:57,eq_bigr_:57,eq_bool:13,eq_class:42,eq_dec:17,eq_ex2:17,eq_ex2_hprop:17,eq_ex2_uncurri:17,eq_ex:17,eq_ex_hprop:17,eq_ex_intro2:17,eq_ex_intro2_hprop:17,eq_ex_intro2_uncurri:17,eq_ex_intro:17,eq_ex_intro_hprop:17,eq_ex_intro_uncurri:17,eq_ex_uncurri:17,eq_ind:[14,27,40],eq_ind_r:[11,27],eq_izr_contraposit:17,eq_map:57,eq_mod_ab:17,eq_mod_opp:17,eq_nat:[24,42],eq_nat_dec:17,eq_nat_equiv:42,eq_pattern:17,eq_rec:[14,27,34,40],eq_rec_r:27,eq_rect:[14,17,27,34,40,67],eq_rect_r:[17,27],eq_refl:[5,9,11,12,13,14,17,27,40,57,64,66,67,71],eq_reflex:59,eq_rel:3,eq_rel_reflex:3,eq_rel_rel:3,eq_rel_symmetr:3,eq_rel_transit:3,eq_set:3,eq_set_refl:3,eq_set_rel:3,eq_set_rel_reflex:3,eq_set_rel_rel:3,eq_set_rel_symmetr:3,eq_set_rel_transit:3,eq_set_sym:3,eq_set_tran:3,eq_sig:[17,67],eq_sigt_rect:17,eq_sind:[14,27,40],eq_sym:[27,40,44],eq_symmetr:59,eq_tran:[27,59],eq_trans_assoc:59,eq_tru:17,eq_true_is_tru:12,eqa:[3,13],eqab:57,eqac:57,eqb0:57,eqb:[3,5,13,17,27,36,59],eqb_correct:36,eqb_leibniz:13,eqb_sym:59,eqba:57,eqblr:17,eqbrl:17,eqca:57,eqd0:57,eqdec:[13,38,60],eqdec_def:13,eqdep:17,eqdep_dec:[17,67],eqlista:17,eqn:[17,40,55,57,58,67,71],eqn_mul1:57,eqnarrai:34,eqnat:[17,26,42],eqnot:17,eqo:3,eqp:57,eqst:30,eqst_hd:30,eqst_tl:30,eqt:[17,46],eqt_ind:46,eqt_rec:46,eqt_rect:46,eqt_sind:46,equal:[3,5,8,10,11,12,13,14,17,24,25,26,30,31,32,34,35,36,39,40,42,44,46,52,54,55,57,58,60,61,65,71,72,77],equalitiesfact:17,equality_intropattern:58,equat:[5,6,14,17,24,25,27,34,40,42,46,53,55,58,60,61,64,67,72],equations_plugin:53,equiconsist:34,equip:[3,4,17,24,27,36,42,64],equiv:[5,34,39],equival:[3,9,11,12,13,14,17,24,25,26,27,28,29,32,34,35,36,37,38,41,42,46,51,52,53,54,55,59,60,62,64,66,67,71,75],equivalence_class:64,equivalence_reflex:[3,59],equivalence_symmetr:[3,59],equivalence_transit:3,equivlista:17,eras:[17,44,57,58,67,75],erasur:[58,67],erbsen:17,erememb:[17,43,58],erewrit:[17,43,64],ergo:17,eright:[17,43,67],erik:17,erika:17,err:[42,55],erron:17,error:[2,3,4,9,10,11,12,13,14,16,17,24,25,27,28,29,32,34,35,37,38,39,40,41,42,44,46,51,52,53,57,58,59,60,62,64,66,67,71,72,75],es:10,esc:17,escap:[12,17,25,51,53,71],eset:[17,43,58],eshkeev:17,esimplifi:67,esimplify_eq:[17,43],especi:[7,15,17,24,26,34,44,46,54,57,60,62,64,71],esplit:[17,43,67],essai:77,essenti:[2,17,25,34,55,57,67,71],establish:[3,17,57],estim:74,et:[3,24,77],eta:[13,17,25,31,37],etc:[2,4,9,14,17,24,25,26,27,33,35,42,44,45,51,52,53,54,55,57,59,71,75],etcdir:17,eth:17,ethan:17,etransit:[3,17,43,64],eucl_dev:2,euclid:[2,17,24],euclid_intro:17,euclid_rec:17,euclidean:[11,17,24,25,57],euclidean_division_equations_cleanup:[5,17],euclidean_division_equations_find_duplicate_quoti:5,euclidean_division_equations_flag:17,eugen:77,european:[24,77],ev:58,eval:[3,5,12,14,17,24,25,27,29,30,31,32,35,37,42,52,53,55,59],eval_bf:5,eval_earli:54,evalu:[2,3,9,11,17,24,25,28,30,34,35,41,53,57,60,64,71],evar:[17,24,54,55,57,58,59,64,71],evarconv:17,evarmap:17,even:[0,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,68,69,70,71,72,73,74,75,76,77],even_0:34,even_:34,even_alt:17,even_alt_even:17,even_even:17,even_ind:[34,67],even_o:34,even_odd:[17,67],even_odd_ind:17,even_sind:[34,67],even_ss:34,eveno:[0,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],event:[2,17,51],event_oddt_dec:17,event_oddt_rect:17,eventu:[5,17,34,42,43,52,54,55,57,58,60,66],ever:[17,52,55,57,67,71],everi:[3,9,11,12,13,14,17,28,29,34,40,51,52,54,55,57,58,64,71],everybodi:17,everyth:[2,17,52,53],everywher:[2,17,55,58,64],evgeni:[5,17],evgenii:17,evolut:[17,77],evolv:[17,24,37,52,54],ex1:55,ex2:[17,24,27,55,67],ex2_ind:27,ex2_sind:27,ex:[3,17,24,27,44,58,67,71],ex_ind:27,ex_intro2:27,ex_intro:[27,37,41,57,60,66],ex_sind:27,exact:[3,12,14,17,24,25,35,40,43,53,54,55,58,59,60,64,66,67,71],exact_no_check:[58,66],exactli:[4,10,11,13,17,26,27,34,40,42,44,46,51,52,54,55,57,59,66,67,71],exactly_onc:25,examin:[46,52,54,66,67,71],exampl:[7,8,9,13,24,25,32,36,45],example_lra:5,example_map:57,exc:[24,27],exce:[59,67],excel:17,except:[2,3,4,11,12,13,14,17,24,25,26,27,29,31,34,35,36,38,40,43,51,52,53,54,57,58,59,60,64,66,67,71,75],exception:[17,24,64],excerpt:36,excess:24,exchang:[24,52,66],exclud:[17,34,41,51,53,54,55,57,59],exclus:[29,57],execut:[6,17,24,25,29,36,51,52,53,55,57,59,64,66,67,71],exempl:24,exfalso:[17,58],exhaust:[17,29,46,53,54,55,59],exhibit:5,exist2:27,exist:[3,4,5,9,11,13,14,17,25,26,27,28,29,31,32,34,36,37,39,41,42,46,51,52,53,54,55,57,58,59,60,63,64,66,67,71,74],existenti:[3,6,9,10,13,17,24,25,26,34,41,45,54,58,59,60,64,66,67],exists2:[17,27,29,57],exists_app:17,exists_concat:17,exists_differ:71,exists_flat_map:17,exists_fold_right:17,exists_foral:17,exists_map:17,exists_non_nul:71,exists_nth:17,exists_or:17,exists_or_inv:17,exists_rev:17,existt2:27,existt:[17,27,67,71],exit:[8,17,25,30,32,34,38,51,52,54,59,60,75],exn:55,exp:57,exp_ineq1:17,exp_ineq1_l:17,exp_intro:34,expand:[2,13,14,17,28,29,30,31,35,37,41,46,52,54,55,57,58,64,67,71],expans:[10,12,13,17,25,34,53,55,57,64,71],expect:[2,3,4,11,12,14,17,24,26,29,31,32,33,34,40,41,42,43,44,46,51,52,54,55,57,58,60,64,67,71],expens:[13,17,54,66],experi:[17,24,51,77],experienc:66,experiment:[5,10,12,14,17,24,51,53,54,62,66,67,71,72],expert:53,expir:24,explain:[8,13,17,24,29,42,51,52,57,60,71,72,74],explan:[3,13,37,45,51,58,59,67],explicit:[9,10,13,17,24,25,28,31,34,37,39,41,46,55,58,60,64,66,67,71],explicit_id:71,explicit_subentri:71,explicitli:[2,4,12,13,14,17,24,27,28,29,34,38,39,43,46,51,52,53,55,57,58,59,60,64,66,67,71,74],exploit:[3,17,24,57,67],explor:[5,17,59],explos:17,expn:57,expon:[11,17,29,71],exponenti:[5,17,29],expos:[2,17,25,40,41,57,71],exposit:17,expr1:54,expr:[17,54,55,71],expr_0:17,expr_1:17,expr_i:17,expr_ind:71,expr_n:17,expr_rec:71,expr_rect:71,expr_sind:71,express:[2,3,4,5,9,10,11,14,17,24,25,26,27,28,29,30,31,32,34,35,39,40,41,43,44,57,58,59,60,64,66,67,75],exprop:34,exprop_ind:34,exprop_sind:34,expung:24,exs_intro:34,exset:[26,34],ext2:[17,24],ext4:51,ext:[17,24,34],ext_intro:34,extend:[3,4,5,9,10,11,14,17,24,25,26,27,28,29,32,34,35,37,40,41,42,45,51,52,53,55,59,60,71,77],extens:[6,9,10,11,12,14,17,25,26,29,32,41,42,52,53,59,62,63],extension:[12,17,27,30,57],extent:[17,71],extern:[2,5,11,13,17,29,33,52,54,55,59,60,63,66,73,74,75],extgcd:17,extocamlnativestr:17,extra:[8,9,17,24,25,30,34,41,42,46,53,54,57,62,64,66,71,75],extra_reifi:17,extra_scop:17,extract:[9,25,26,27,29,34,36,51,53,57,59,71,72,73,77],extraction2002:77,extraction_plugin:[2,9,34,57,72],extractor:[17,24],extran:[17,52],extrem:[14,17,29,57],extrhaskellbas:17,extrhaskellstr:17,extrocaml:17,extrocamlbigintconv:17,extrocamlfloat:36,extrocamlint63:[17,36],extrocamlintconv:2,extrocamlnatbigint:17,extrocamlnatint:2,extrocamlnativestr:17,extrocamlparrai:36,extrocamlpstr:36,extrocamlstr:17,extrocamlzbigint:17,extyp:34,extype_ind:34,extype_rec:34,extype_rect:34,extype_sind:34,f0:[34,57,67],f10:52,f11:52,f1:[13,17,41,51,57,71],f2:[17,41,51,52,55,57],f4:52,f8:52,f9:52,f:[0,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],f_1:[11,34],f_1_neq_0:11,f_2:[11,34],f_:24,f_equal2:27,f_equal2_plu:59,f_equal3:27,f_equal4:27,f_equal5:27,f_equal:[17,27],f_equalx:17,f_ext:27,f_i:34,f_impl:2,f_ind:58,f_inj:34,f_j:34,f_k:34,f_l:34,f_n:34,f_r:11,f_rec:58,f_rect:58,f_scope:71,f_sind:58,fabian:17,face:[3,17,75],facil:[13,17,24,52,54,55,57,59],facilit:[17,51,57],fact:[2,5,11,14,17,24,28,32,34,39,41,42,46,54,55,57,58,62,64,66,67,71,75],factor:[2,5,11,17,25,34,45],factori:[17,24,54,55,64],factoriz:[17,46],fail:[2,3,4,5,8,9,10,12,13,14,17,24,25,26,29,30,34,35,40,41,42,43,44,52,53,55,58,59,60,62,64,66,67,71,72,75],failur:[3,8,13,14,17,24,25,46,53,55,57,59,60,62,64,71,77],fairli:[17,57],faithful:17,faithfulli:13,fake:60,fall:[3,9,10,13,24,53,58],fals:[2,4,5,9,10,12,13,17,24,27,34,37,40,41,43,46,51,54,55,57,58,59,62,64,66,67,71],false_rec:27,false_rect:46,falsiti:54,falso:[17,58],famili:[4,14,17,24,25,34,40,54,55,63,67,71],faq:17,far:[11,24,46,52,57,66,71],farka:17,farzon:17,fashion:[17,24,51],fast:[3,17,24,25,53],fast_:17,fast_integ:17,faster:[11,17,24,51,58,59,62,64],fastest:53,fatal:[17,25,57],fault:[2,24,71],favor:[17,41,51],fcomp:41,fct:4,fct_of_incr_fct:4,fd:34,fdiv_def:11,fear:33,featur:[2,3,8,11,17,24,25,29,32,33,35,36,44,46,51,52,53,54,55,57,59,66,71,72,73,74,76],feb:24,februari:[17,24],fed:[9,17,55],feed:60,feedback:[8,17],feel:52,feferman:24,fehrl:17,fei:77,felti:24,feq:27,fermat:52,fernandez:17,fernando:17,fetch:66,few:[2,3,17,24,27,29,34,35,36,37,51,52,53,55,57,58,71,73,75],fewer:[17,51,58,64,66],ff:5,ffi:[17,25,55],fg:4,fgt:27,fi:13,field:[4,5,7,12,13,14,17,24,25,27,42,51,53,55,59,61,74],field_mod:11,field_simplifi:17,field_simplify_eq:17,field_spec:37,field_theori:11,field_val:[13,37],fieldnam:37,fifth:17,figur:[52,57],file1:[52,53],file2:[52,53],file:[2,3,5,6,7,8,9,11,17,24,25,27,29,34,35,36,41,42,43,54,55,57,58,60,64,66,71,72,73,76],filen:52,filenam:[14,17,25,51,52,59,64,75],filesystem:[53,59],fill:[2,9,13,17,25,52,55,57,62,71],filliatr:[24,77],filter:[13,17,30,51,53,59,60],filter_2_4:46,filter_app:17,filter_fals:17,filter_length:17,filter_length_forallb:17,filter_length_l:17,filter_map_swap:17,filter_rev:17,filter_some_square_corn:46,filter_tru:17,filtered_import:[17,35,59],filteropt:51,fin:[17,71],fin_scop:71,find:[2,3,4,5,7,11,13,14,16,17,25,27,29,34,42,43,51,52,53,54,55,57,58,59,62,64,66,67,71,72,77],find_duplicate_quoti:17,findlib:[17,53,59],fine:[17,41,51,52,57,64],finer:[2,17,34,57],finfun:17,finish:[8,13,17,29,46,54,60,64,66,67],finish_tim:[17,54],finit:[3,5,17,24,27,30,34],finite_alt:17,finite_dec:17,finv_l:11,fire:[2,14,17],firefox:52,first:[2,4,5,6,8,9,11,13,14,15,17,24,25,26,27,35,37,38,40,41,42,43,44,51,52,53,55,58,59,60,62,64,65,66,67,71,72,74,75,77],first_lett:29,firstn:17,firstn_length:17,firstord:[17,29,62],fissor:17,fit:[14,17,27,29,34,52,55,57,71],five:[17,27,64],fix:[0,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,32,33,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],fix_decl:[34,57],fix_definit:[34,38,72],fix_eq:[17,27],fix_f:27,fix_f_eq:27,fix_f_inv:[17,27],fixabl:17,fixannot:[9,34,72],fixpoint:[2,3,10,13,17,24,25,27,29,30,31,32,37,38,41,44,46,52,57,59,64,66,67,71,72],fk:57,flag:[2,4,5,8,9,10,12,13,14,16,24,25,27,32,34,35,37,38,40,41,43,44,46,51,52,53,54,55,57,58,60,62,64,66,67,71],flagship:25,flambda:17,flat_map:[17,24,27],flat_map_app:17,flat_map_constant_length:17,flat_map_ext:17,flat_map_length:17,flatten:17,flavor:[17,37,71],fledg:17,flexibl:[14,17,55,58,64],flh:5,flip:[3,17],float64:36,float64_mul:36,float64_typ:36,float_class:27,float_comparison:27,float_scop:[27,36],floataxiom:17,floatlemma:17,floatop:[17,36],flocq:27,floor:17,florath:17,florent:17,florin:17,flow:25,flt:27,fly:[17,55,57],fm:13,fmap:[17,60],fmapavl:17,fmapfullavl:17,fmapintmap:17,fn:51,fnotcompar:27,fo:2,focu:[17,24,34,43,54,55,57,66,67],focus:[6,17,25,43,55,57,58,59,60],fof:14,fold:[3,17,37,57],fold_left2:17,fold_left:[17,27],fold_left_length:17,fold_left_rev_right:17,fold_left_s_o:17,fold_right2:17,fold_right:[17,27],fold_right_shiftin:17,foldabl:17,folder:[17,52,53],follow:[2,3,4,5,6,8,9,11,12,13,14,17,24,25,26,27,28,29,30,33,34,35,36,37,38,40,41,42,43,46,51,52,53,54,55,57,58,59,60,62,64,66,67,71,72,74,75],fondamental:77,font:[17,52,53,75],foo0:[53,55],foo1:53,foo:[2,11,14,17,29,35,38,40,43,51,52,53,55,57,58,59,64,66,71,74,75],foo_ind:[12,17,57],foo_rec:17,foo_rect:17,foo_sind:12,foo_subproof:38,foobar:14,foolib:17,footnot:[11,38,57,71],footprint:17,fop:5,for_all2:17,for_each_go:[54,55,71],foral:[2,3,4,5,6,7,9,10,11,12,13,14,17,25,26,27,29,30,31,32,34,36,37,41,42,43,44,46,52,54,55,57,58,59,60,62,64,66,67,71,72,75],forall2:17,forall2_append:17,forall2_cons_iff:17,forall2_flip:17,forall2_impl:17,forall2_length:17,forall2_nil:17,forall2_nth:17,forall2_nth_ord:17,forall2_refl:17,forall_and:17,forall_and_inv:17,forall_app:17,forall_append:17,forall_concat:17,forall_cons_iff:17,forall_elt:17,forall_eq_repeat:17,forall_exists_exists_forall2:17,forall_flat_map:17,forall_fold_right:17,forall_foral:17,forall_imag:17,forall_impl:17,forall_map:17,forall_nil_iff:17,forall_nth:17,forall_nth_ord:17,forall_rev:17,forall_shiftin:17,forallb_filt:17,forallb_filter_id:17,forbid:40,forbidden:[12,17,24,25],forc:[4,8,11,17,24,34,42,44,52,53,54,57,60,64,66,67,71],force2:71,ford:17,foreground:66,foreign:[2,17],forese:24,forest:[0,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,68,69,70,71,72,73,74,75,76,77],forest_ind:[34,67,72],forest_rec:[34,67,72],forest_rect:[34,67,72],forest_s:[34,72],forest_sind:[34,67,72],forest_size_equ:72,forest_size_ind2:72,forest_size_ind:72,forest_size_rec:72,forest_size_rect:72,forest_tree_ind:67,forest_tree_rec:67,forest_tree_rect:67,forg:51,forget:[4,11,37,55,59,60,67],forgot:[32,71],forgotten:4,fork:17,form:[2,3,4,5,6,7,9,11,13,17,24,25,26,27,28,29,30,31,32,35,37,38,39,40,42,43,44,46,51,52,53,54,55,57,58,59,60,62,64,66,67,71,72,75],formal:[4,6,10,17,24,25,26,29,31,32,34,37,39,41,51,55,57,67,77],formalis:[24,57,77],format:[14,17,24,26,27,35,37,42,51,52,53,57,71,75],formatt:59,formel:24,former:[17,29,30,57,75],formerli:17,formul:[17,42],formula:[5,7,26,57,58,62,77],forster:17,forth:[25,50,57,60],forthcom:17,forum:17,forward:[17,24,52,53,57,62,66],found:[2,4,5,9,11,13,17,25,29,30,34,35,36,38,39,42,46,51,54,55,57,58,59,62,64,67,71,72,75],foundat:[17,24,29,54,57,77],founded:[17,24],founifi:2,four:[8,17,25,34,52,54,55,57,71],fourier:[17,24],fourth:[17,54,57],fr:[17,24,25,27,53,75,77],frac:[17,26,31,34,35,38],fraction:[7,11,17,24,27,29,37,57,71],fragil:[17,54,57,59,60,63,66],fragment:[55,57,71],frame:[17,52],framework:[2,17,24],franc:[24,77],francoi:17,frank:[17,77],free:[11,17,24,26,34,44,52,54,55,57,58,62,64,71,75,77],freedom:17,freek:24,freeli:[14,57],freez:13,frege:24,freiburg:77,french:17,frequenc:17,frequent:[11,17,25,53,57,66,67,71],fresh:[3,14,17,24,25,31,34,53,57,58,64,66,67,71],freshid:17,freshnamespac:40,freund:24,frexp:17,frexp_spec:17,frh:5,friendli:[17,24,52],frii:17,fring:17,from:[2,3,4,5,6,8,9,10,11,12,13,14,17,24,25,26,27,28,29,30,31,34,36,37,38,39,40,41,42,43,46,51,52,53,54,57,58,59,60,62,63,64,66,67,71,72,73,75,77],front:[57,59],frozen:24,frshiftexp:27,fs:[2,71],fset:[17,27,60],fsetavl:17,fsetdecid:17,fsetfullavl:17,fsetinterfac:17,fsetproperti:17,fst:[17,24,27,35,42,46,71],fst_list_prod:17,fta:24,ftorradix:8,ftp:77,fubar:57,fulfil:[2,17,67],full:[13,14,17,24,25,30,34,43,46,52,57,58,64,66,71,77],fuller:24,fullfil:17,fullgrammar:71,fulli:[2,3,8,17,24,26,28,31,32,35,38,44,51,52,53,54,55,58,59,64,66,71,72],fun:[2,3,4,5,6,9,10,11,12,13,14,17,25,26,27,29,30,31,32,34,35,37,38,40,41,42,43,44,46,54,55,57,58,59,64,66,67,71,72,75],fun_scop:17,funapp:71,func_scheme_def:72,funclass:[4,17,41,71],functin:17,function_scop:[14,17,25,34,46,57,67],functions_in_zfc:24,functor:[0,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,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],functor_app_annot:35,functori:17,fund:17,fundament:[17,24,31,57],funext_down:14,funext_typ:14,funind:[17,57,59,72],funind_plugin:[57,72],further:[3,17,27,30,35,41,51,52,54,55,57,64,66,67,71],furthermor:[10,17,24,25,26,29,31,33,34,51,52,55,57,63,66],futur:[4,9,10,13,14,17,32,34,41,51,52,53,57,62,66,71,77],fuzz:17,fv:11,g0:[60,67],g1:60,g2:60,g:[3,4,5,9,10,13,14,17,24,27,28,29,30,31,34,35,36,41,43,44,46,52,53,54,55,57,58,59,60,62,64,66,67,71,75,77],g_1:57,g_:57,g_equat:53,g_i:34,g_n:57,ga:77,gabriel:17,gadt:2,gain:[17,24],gallego:17,gallina:[11,17,25,27,41,66,75],gamma:[0,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],gan:17,gap:57,gappa:17,garbag:[17,75],gariano:17,garillot:17,garrigu:17,gather:[17,24,27,55,57,58],gave:[17,24,58],gc:[17,66],gcd:[17,59],gcd_comm:59,gcd_mod:17,gcd_mod_l:17,gcd_mod_r:17,gcd_mul_diag_l:17,gcd_uniqu:17,gcd_unique_alt:17,gcst19:[12,39,77],gdk_use_xft:52,ge:[5,17,27],gear:[8,52],geb:5,geb_g:17,gen:57,gen_constant_modul:17,gen_item:57,gen_x:67,genarg:52,gener:[5,7,8,9,12,13,16,17,24,25,27,28,30,31,32,34,35,36,37,38,39,40,43,46,51,52,53,58,59,60,61,62,64,66,75,77],generalis:57,generaliz:[13,17,44],generalize_eq:67,generalize_eqs_var:67,generalizing_bind:[28,44],generer:17,genericminmax:17,genral:17,geometri:[7,24],geoproof:17,georg:[17,57,77],georgian:29,germani:77,get:[2,5,9,11,13,14,17,24,25,27,28,29,34,36,42,51,52,53,55,58,59,60,64,66,67],get_current_context:17,get_set_oth:36,get_set_sam:36,get_sign:11,gett:37,getter:17,geuver:24,gexpn0:57,gexpn1:57,gexpn_add:57,gfail:[17,54,60],ghc:17,giana:17,gianfranco:77,giarrusso:17,gift:[24,77],gilbert:[17,77],gill:[24,72],gimenez94:[34,77],gimenez95:[30,77],gimenez98:[30,77],gimenezcasteran05:[30,77],gintuit:17,giovini:77,girard:[24,77],gist:17,git:[17,53],github:[2,5,17,51,52,71],gitlab:17,gitter:17,give:[2,3,4,5,7,8,9,11,13,14,17,24,25,26,27,28,29,31,32,34,35,37,40,41,42,45,46,51,52,53,54,55,57,58,59,64,66,67,71,75],give_up:17,given:[2,3,4,5,9,10,11,13,14,17,24,25,27,28,29,32,35,36,37,40,41,42,43,44,46,51,53,54,55,57,58,59,60,62,64,66,67,71,72,74,75],glanc:57,glob:[17,24,51,75],glob_constr:55,glob_term:17,global:[2,3,4,5,9,13,17,24,25,26,28,29,31,32,34,35,37,38,39,41,42,44,51,53,55,57,58,59,60,62,64,66,67,75],globalis:24,globfil:53,glondu:17,gloss:37,glossari:[16,17,25,29],glt89:[66,77],glu:3,gmatch_hyp_pattern:55,gmatch_pattern:55,gmatch_rul:55,gmn:[7,77],gmp:17,gnu:[17,51,53],go:[2,5,9,17,24,30,42,51,52,54,55,57,59,60,64,67,71,75],goal0:[6,43,58,66],goal:[3,6,7,8,9,12,13,14,17,24,25,27,29,31,34,35,36,37,38,42,43,44,52,53,59,60,61,62,64,71,72,74],goal_match_list:55,goal_occurr:58,goal_pattern:54,goal_selector:54,goal_tact:54,goe:[17,53,55,59,66],goir:77,gone:17,gonthier:[17,57,77],good:[11,17,53,54,55,57,66],googl:[51,53],got:[17,34,67],gothenburg:77,gothic:29,gotten:52,goubault:24,govern:[17,41,44,52,67],gr:77,grab:17,gradual:[17,58],grai:[29,52],grain:[2,17,41],grammar:[10,17,25,28,29,54,55,57,58,62,71],grant:17,granular:[52,55],graph:[2,14,17,24,25,39,54,72],graphic:[17,25,29,51,52],graphviz:[14,17],grasp:57,grate:17,grayson:17,great:[31,64],greater:[14,17,24,34,52,71],greatli:[17,24],greek:[17,29,75],green:[17,29,52,66],greg:17,gregersen:17,gregoirel02:[64,77],gregori:17,grep:59,grinberg:17,groebner:17,groot:77,gross:17,ground:[14,17,54,62,71,75],group:[2,4,17,24,37,42,52,53,54,57,58,60],grow:[24,54,55,59],growth:54,gruetter:17,gruin:17,grundlagen:24,gt:[17,27,42],gt_wf_rec:2,gt_wf_rect:17,gtb:5,gtb_gt:17,gtk2:17,gtk3:17,gtk:[17,52],gtk_accel_path:52,gtk_csd:17,gtk_theme:52,gtksourceview:[17,52],guarante:[4,14,17,51,52,53,55],guard:[17,24,25,27,30,32,34,41,44,46,57,59,64,66,67,71,72,77],guarded:[9,66],guess:[2,4,11,17,32,43,53,57,67],gui:[24,52,76],guid:24,guidelin:17,guillaum:17,gulp:66,gv:[14,17],gwhy:17,gyesik:77,gz:[17,51,53],gzip:53,gznd11:[42,77],h0:[54,55,57,58,62,64,66,67],h1:[11,17,34,43,54,55,57,58,62,66,67],h23:57,h2:[17,34,43,54,55,57,58,67],h2_0:67,h2_:67,h3:[58,67],h:[3,4,6,9,11,12,13,14,17,24,27,34,40,44,46,51,54,55,57,58,62,64,66,67,72,75,77],ha:[2,3,4,5,6,8,9,11,12,13,14,17,24,25,26,27,28,29,30,31,32,34,35,36,37,38,39,40,41,42,43,44,46,51,52,53,54,55,57,58,59,60,62,63,64,66,67,71,72,73,74],haan:17,haani:17,had:[9,13,17,24,42,53,54,55,66],hal:77,half:[17,24,37,66],hallberg:17,hand:[3,10,12,13,17,25,27,29,33,35,52,53,54,55,57,58,64,67,71,72],handi:[17,71],handl:[2,3,8,9,11,17,24,26,37,43,46,53,55,57,58,59,61,62,66,67,71],hangul:29,hao:17,happen:[2,4,9,10,13,17,34,38,46,52,54,55,57,58,64,71,72],hard:[17,55,59,64],hardcod:17,harder:[4,17,58],hardwar:[2,8,24],harm:34,harmless:[34,51],harrison:5,harsh:17,harvei:17,has_evar:17,hash:17,haskel:[2,13,17,24,25,57,64,77],hasn:35,have:[2,3,4,5,7,8,9,10,11,12,13,14,17,24,25,26,27,28,29,30,31,32,33,34,35,36,37,39,40,41,42,43,44,46,51,52,53,55,58,59,60,62,64,66,67,71,73,75],haven:[52,54],hayashi:24,hb:[57,58],hd:[17,30,34,57,72],hd_error_skipn:17,he:[11,17,24,57],head:[3,10,13,14,17,24,26,27,30,35,41,42,44,53,54,55,57,58,59,60,64,67,71],headconcl:[17,59],header:[17,51,75],headhyp:[17,59],heap:[17,54,66],heap_word:66,heapsort:[17,24,27],heart:33,heavi:2,heavili:17,hebb:17,hebrew:[17,29],heel:54,heidelberg:77,heiko:17,held:24,helg:17,helm:[17,24],help:[2,3,8,13,14,15,16,17,24,25,27,29,41,46,51,52,53,54,55,57,58,60,62,67,75],helper:[25,59],henc:[2,3,4,5,8,9,13,14,17,26,34,37,42,51,53,54,57,58,64,67,71],hendrik:17,henk:24,henri:[17,24],heq:[17,54,67],heq_n0:9,heq_n:9,heql:67,heqp:67,her:24,herbelin:[17,24,46],here:[2,3,4,5,9,11,13,14,16,17,24,27,29,31,33,34,35,37,38,41,42,44,46,51,52,53,54,55,57,58,59,60,64,66,67,71,75],hereaft:[26,30,55,57],herm:17,herman:24,heterogen:[17,67],heurist:[2,5,14,17,55,57,58,66],hex:17,hex_int_scop:71,hex_n_scop:17,hex_nat_scop:71,hex_positive_scop:17,hex_uint_scop:71,hex_z_scop:17,hexa:71,hexadecim:[17,27,29,36,52,59],hexdigit:29,hexnat:29,hf:[34,51],hfg:57,hget_evar:17,hi:[17,24,34],hid:17,hidden:[17,24,25,27,53,57,71,75],hidden_arrow:12,hide:[17,25,34,41,44,57,58,66,71],hierarch:[24,35],hierarchi:[14,17,24,25,34,39,51],high:[14,17,24,25,35,59,60,66,72],higher:[3,14,17,24,25,27,40,51,54,57,58,59,60,64,67,71,73,77],highest:71,highli:[10,43,60,63],highlight:[17,51,52,53,57,63,66],higman:2,hijack:17,hilbert:[5,7,17],hinder:17,hindlei:[55,77],hindranc:54,hint:[3,13,14,17,24,25,27,35,38,54,62,64,75],hint_info:[13,60],hintbas:[55,60],hintdb:[13,17,55,60],hints_regexp:60,hiragana:29,histor:[17,25,44,55],histori:[17,25,26,53,59,66],hivert:17,hl:67,hloc:58,hlt:27,hn:66,hnat:44,hnf:[17,24,41,42,57,58,64,67],hnm:57,ho:[17,29,58],hoc:[2,3,17,71,77],hoist:17,hol:5,hold:[3,4,17,30,34,35,40,42,55,58,75],hole:[9,13,17,24,25,40,43,46,55,57,58,59,62,66,67,71],holland:77,home:[17,51,52,53],homebrew:17,homogen:[3,17],homotopi:17,honor:[2,17,51,57,71],honour:57,hood:[5,17],hook:[17,53],hope:[24,52],hopefulli:[17,55],horizont:[17,29,53,71,75],horror:25,host:17,hott:[17,40],how80:[26,66,77],how:[2,7,8,13,17,24,25,27,29,30,34,35,37,42,43,45,51,53,54,57,58,59,60,62,64,67,71,72,74,77],howard:[24,26,66,77],howev:[3,4,5,9,12,13,14,17,24,27,29,34,36,37,41,43,44,46,51,52,53,54,55,57,58,64,66,67,71,72],hp:[57,67],hpa:57,hpb:57,hq:[57,67],hqa:57,hqab:57,hrec:57,hresolve_cor:17,hspace:[26,31,34,35,38],html:[17,25,29,53],http:[2,5,17,24,25,27,50,51,52,53,59,64,71,75,77],hue88:[24,77],hue89:[24,66,77],huet:[24,77],hug:17,huge:[8,11,17,54,57,66],hugo:[17,24,46],hugunin:17,human:[17,25,58,75],hundr:[11,64],hur:17,hv:71,hx:[12,57,58],hy:58,hybrid:17,hydra:2,hyp0:57,hyp:[17,24,55,57,59,66,71],hyp_occ:58,hyp_valu:17,hyperlink:[17,25,29],hypertextu:24,hyphen:74,hypid:58,hypothes:[3,5,9,13,17,24,25,28,32,34,51,57,60,62,64,67,71],hypothesi:[3,9,11,17,24,25,27,28,29,34,38,55,57,59,60,62,64,66,67,71,72,75],hz:54,i1:[34,71],i2:71,i:[0,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],i_1:[7,11,34,35],i_2:[11,57],i_:[3,34,57],i_block:57,i_i:35,i_ind:[46,71],i_item:57,i_j:[34,35],i_k:[7,34,35],i_l:34,i_n:[11,57],i_not_i:34,i_p:34,i_pattern:57,i_rec:[46,71],i_rect:[46,71],i_sind:[46,71],i_view:57,ia:17,icfp:77,icon:[17,52],id0:14,id1:17,id:[3,4,9,10,14,17,24,26,34,35,42,44,51,52,53,54,55,57,58,64,66,71,75],id_1:17,id_fct_funclass:4,id_n:17,id_rew:10,id_str:71,iddec:53,idea:[11,17,34,42,54],ideal:7,idem:24,ident0:51,ident1:51,ident:[2,3,5,6,9,10,11,12,13,14,17,24,25,27,28,29,30,31,32,34,35,37,38,40,43,44,46,51,53,55,57,58,59,60,62,64,66,67,71,72,73,74],ident__i:6,ident_decl:[4,9,13,28,30,32,34,37,38,40,42,59],ident_or_anti:55,identifi:[2,3,9,14,17,24,25,28,29,30,31,35,38,40,41,43,44,46,51,52,53,54,55,57,58,60,66,67,72,75],identityt:17,ideograph:29,idiom:[17,54,55,57,66],idl:52,idn:17,idp:57,idtac:[14,17,25,52,55,57,60,66,71,74],idx:57,ieee:[17,36,77],iempti:71,if_then_els:[17,71],ifeq:53,iff:[3,17,26,27,31,57,59,71],iff_reflex:59,iff_symmetr:59,iff_tran:17,ifflr:57,iffrl:57,ifft:17,ifi:17,igler:17,ignat:17,ignor:[4,13,14,17,24,27,29,31,34,35,44,51,52,53,54,57,58,60,64,66,71],ih:67,ihl:67,ihm:57,ihn0:[67,72],ihn:[57,66,67],ihp:67,ihterm:67,ihu:57,ihv:57,ik:17,ikebuchi:17,ikfprintf:17,ill:[2,4,9,10,17,24,30,34,51,55,64,71,72],illeg:4,illtypedinst:17,illustr:[5,17,34,46,57,60,64],imag:[3,11,17,24,51,52,66],imai:17,imedi:60,immedi:[17,24,27,54,55,57,58,59,60,66],immediatli:17,immut:36,impact:[2,17,53,66,71],imped:54,imper:[17,24,55],impl:[3,5,59],impl_reflex:59,implb:[5,17,27],implb_andb_distrib_r:17,implb_contraposit:17,implb_curri:17,implb_false_iff:17,implb_false_l:17,implb_false_r:17,implb_negb:17,implb_orb_distrib_l:17,implb_orb_distrib_r:17,implb_sam:17,implb_true_iff:17,implb_true_l:17,implb_true_r:17,implement:[3,8,11,12,13,17,24,25,27,29,34,35,36,37,39,43,46,54,55,57,58,59,60,62,64,66,67,71,72,77],implementor:59,impli:[2,3,10,14,17,24,30,34,57,67,71],implic:[3,17,26,27,28,42,54,57,60,66,67,71],implicit:[2,3,5,9,13,17,24,25,28,33,34,37,38,42,43,45,51,53,55,57,58,59,66,67,75],implicit_bind:[28,44],implicitli:[3,13,14,17,24,34,51,55,60,64],implict:41,implypp:17,import_categori:[17,35,59],importantli:17,impos:[24,30,34,57],imposs:[5,17,34,46,53,58,67],impract:53,impred:[2,12,14,17,24,25,34,51,53,77],improp:17,improv:[2,3,8,11,17,24,29,52,54,57,67],inE:17,in_concat:17,in_cons_iff:17,in_context:17,in_dec:17,in_elt:17,in_elt_inv:17,in_flat_map_exist:17,in_goal:17,in_hd:67,in_hyp_a:58,in_iff_nth_error:17,in_in_remov:17,in_inj_comp:17,in_left:17,in_nth:17,in_remov:17,in_rev:17,in_right:17,in_shiftin:17,in_tl:67,inabl:64,inaccess:17,inact:66,inadvert:[17,52],inc:17,incant:57,incident:17,incl:[17,59],incl_app_app:17,incl_app_inv:17,incl_cons_inv:17,incl_exist:17,incl_filt:17,incl_foral:17,incl_forall_in_iff:17,incl_l_nil:17,incl_map:17,incl_nil_l:17,incl_refl:59,inclass:17,includ:[2,3,5,8,9,12,13,14,17,24,25,27,28,29,34,35,36,38,39,40,41,43,44,51,52,53,54,55,57,59,60,62,64,66,67,71,73,75],include_subdir:53,inclus:[14,17,54,55],incoher:[17,46],incom:[4,17],incompar:71,incompat:[14,24,25,34,41,46,57,59,66,71],incompatibili:17,incompatibilit:24,incomplet:[5,8,10,17,24,46,58,66,67,71],inconsist:[2,8,10,12,14,17,24,26,34,39,44,51,59,66,67,71],incorrect:[2,8,12,14,17,25,34,37,46,52,57,66],incorrectli:[12,17,55],incr_fct:4,increas:[3,5,8,17,24,53,57,62],incred:55,increment:[17,24,30,31,32,33,34,38,55,66],incur:[17,66],ind1:35,ind2:35,ind:[0,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],ind_bool:59,indag:77,inde:[3,4,11,12,13,14,17,25,26,29,30,34,35,40,41,42,43,44,46,53,54,55,57,58,60,64,66,67,71,72],indefclass:17,indefinit:17,indefinitedescript:17,indent:[8,17,25,66,71,75],independ:[2,13,14,17,24,34,51,52,53,54,55,57,67],indetermin:57,index:[3,13,17,24,25,26,27,29,39,40,44,52,58,60,64,66,67,73,75],index_iota:57,indic:[2,8,11,12,13,14,17,24,26,31,34,35,39,40,41,42,43,46,51,52,53,54,57,58,59,62,64,66,67,71],indirect:[17,64],indirectli:[17,24,58,59,60,74],indistinguish:[14,37],individu:[17,53,55,64,67,71],indp1:35,indp2:35,indp:[0,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],indpstr:[0,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],indrec:17,induc:[17,24],induct:[4,5,9,10,11,12,13,14,17,24,25,27,29,30,31,32,33,35,37,41,42,44,52,54,55,57,58,59,60,62,64,65,66,73,75,77],induction_arg:[55,67],induction_claus:[55,67],induction_ltof1:17,induction_ltof2:2,induction_principl:67,induction_test2:67,induction_test:67,inductive_definit:[30,34],ineffici:[5,17,24,57],inequ:[5,17,24,60],inexact:27,infam:17,infer:[3,4,9,10,13,14,24,25,26,34,37,40,41,42,45,46,51,57,58,60,62,67,71],infin:[27,30,71],infinit:[12,27,30,34,39],infinite_loop:34,infix:[2,14,17,24,25,27,42,57,58,64,74],inflat:17,influenc:[17,24,34],info:[5,17,54,60],info_auto:[17,60],info_eauto:[17,60],info_trivi:17,infoh:54,inform:[2,3,4,10,12,13,14,17,24,25,26,27,29,30,34,37,39,41,42,43,44,46,51,52,53,54,55,57,58,59,60,62,64,67,72,75,77],informatiqu:[24,77],infrastructur:[3,25,42,53],ing:[17,74],ingredi:54,inhabit:[14,29,31,32,34,37,40,43,46,51],inher:57,inherit:[17,24,25,42,52,55],inhibit:[17,57],ini:52,init:[9,14,17,27,28,35,51,54,55,58,59,60,66,67,71],initi:[2,6,7,11,13,17,24,27,29,38,46,52,53,54,55,57,58,59,60,62,63,64,66,67,71,74,75],initialr:11,inj:62,inj_compr:17,inj_land:17,inj_ldiff:17,inj_lor:17,inj_lt:57,inj_lxor:17,inj_shiftl:17,inj_shiftr:17,inject:[0,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],inject_nat:17,injective_map_nodup_in:17,injtyp:[5,17],inl:[27,40,57],inleft:27,inlin:[17,24,25,28,35,64,66,72,75],inner:[2,14,17,35,42,43,54,55,57,59,62,64,66,67,71,75],innermost:[54,71],input:[3,4,9,10,14,17,25,27,29,35,44,46,51,54,57,58,60,64,71,72,74,75],inputenc:75,inr:[17,27,40],inr_0:17,inr_1:17,inr_archim:17,inr_izr_inz:17,inr_unbound:17,inria:[17,24,25,27,53,75,77],inright:27,ins:[17,58,59],insarov:17,insensit:17,inser_trans_r:17,insert:[3,4,9,12,13,17,24,25,29,41,46,52,53,55,57,66,71,75],insid:[2,3,4,8,9,13,14,17,24,25,28,29,34,35,38,46,52,55,57,58,59,60,64,66,67,71,74],insofar:55,inspect:[2,17,57,59],inspir:[17,24,75],inst:37,instabl:17,instal:[17,25,27,35,51,52,64,66,72,73],installcoqdocroot:17,instanc:[2,3,4,5,10,11,12,14,17,25,26,27,28,29,30,31,34,35,36,37,38,39,40,41,42,44,46,51,52,53,55,57,58,59,60,62,64,66,67,71,75],instancenam:13,instanti:[3,10,13,14,17,24,34,35,43,44,54,55,57,58,60,62,67,71],instantiate_ltac_vari:58,instantli:57,instat:42,instead:[2,3,4,7,8,11,12,13,14,17,24,26,28,33,34,35,36,37,43,44,46,51,52,53,54,55,57,58,59,60,62,64,66,67,71,72,74,75],institut:[24,27],instruct:[2,5,17,53,58,59],instrument:61,insub:57,insubt:57,insuffici:[14,17,51],insur:24,int31:17,int63:[17,71],int63_eq:[36,59],int63_typ:[36,59],int63not:17,int_mult:57,int_of_nat:2,int_or_var:[3,54,66,71],int_part_frac_part_spec:17,int_part_spec:17,int_scop:17,int_wrap:71,int_wrapp:71,intead:17,integ:[2,3,7,11,14,17,24,25,29,34,39,52,53,54,55,57,59,60,64,66],integr:[10,11,17,24,25,27,51,52,57,61,73],intellig:[24,42],intend:[3,17,24,28,32,39,51,57,64,66,71],intens:[11,17,24,64],intent:[17,24,28,57],intention:51,intepret:17,inter:[24,53],interact:[3,10,13,17,24,25,32,33,37,38,40,42,43,52,59,65,66,67,75,76,77],interchang:[53,66],interdepend:25,interest:[2,4,5,11,17,24,31,42,54,57,67],interfac:[2,17,24,25,35,52,53,66,74,75,76],interfer:[57,71],interleav:[11,17,58],intermedi:[17,27,57,66],intermediari:[2,64],intern:[3,5,11,14,17,24,25,31,34,37,44,51,53,54,55,58,60,62,66,67,71,72,73,74,77],internal_:59,internet:52,internship:24,interpet:58,interpol:[17,53,75],interpret:[3,5,9,11,13,17,24,25,27,29,32,34,35,41,44,51,52,53,54,55,59,75],interrupt:[17,52,54,59],intersect:9,intertwin:[17,57],interv:52,intervent:52,intf:17,intmap:[17,24],intric:[54,55],intro:[3,5,11,12,13,17,24,25,27,34,42,43,44,52,54,55,60,62,64,66,67,71,72],introa:34,introduc:[3,5,8,10,11,13,14,17,24,25,28,30,31,34,35,37,38,43,44,46,51,52,55,57,58,59,60,62,66,67,71,72,75],introduct:[7,13,17,24,30,34,62,67,71],introl:58,intron:57,intronf:57,introntf:57,intropattern:[17,55,58,67],intror:58,intros_until:55,intuit:[4,11,17,24,29,55,58,62],intuition_solv:[17,62],intuitionist:[17,24,25,27,34,57,62,77],intuitionnist:77,inv_high:14,inv_low:14,invalid:[17,24,40,52,54,59,64,66,71],invalid_argu:[17,55],invari:[14,17,55],invariant_ind:14,invariant_rec:14,invariant_rect:14,invariant_sind:14,invers:[3,11,17,24,25,27,31,58,60,64,72,77],inverse_imag:17,inversion_clear:67,inversion_sigma:17,invert:[13,17,57,67,72],invert_con:67,investig:[17,24,77],invis:[17,53,57],invit:[24,42],invoc:[25,53,54,57,59],invok:[11,17,34,51,53,59,60,66,67,75],involv:[3,4,9,12,17,24,25,26,34,41,42,51,52,53,54,57,59,60,62,64,67],inz:17,io:[17,25],iota:[0,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],ip_i:34,ipat:[17,57],ipattern:17,ipr_2_xh:17,ipr_2_xi:17,ipr_2_xo:17,ipr_eq:17,ipr_ge_1:17,ipr_gt_0:17,ipr_ipr_2:17,ipr_l:17,ipr_lt:17,ipr_not_1:17,ipr_xh:17,ipr_xi:17,ipr_xo:17,irif:77,irr_high:14,irr_low:14,irreduc:[17,37,64,71],irrefut:[17,25,32,40,57],irrelev:[14,17,25,32,33,34,39,54,55,57,64,77],irrelevant_ind:14,irrelevant_rec:14,irrelevant_rect:14,irrelevant_sind:14,irrevers:[17,24,64],irst:77,is_arrai:17,is_clos:17,is_conj:54,is_const:17,is_constructor:17,is_double_moins_un:17,is_empti:17,is_evar:[17,54],is_float:17,is_ind:[17,54],is_law:42,is_law_:42,is_proj:17,is_tru:[12,57],is_true_eq_tru:12,is_uint63:17,is_zero:46,isaac:17,isbn:77,island:77,islezero:17,isn:[9,10,17,28,52,57,58,60,64,66,67],iso:[17,75],iso_axiom:54,isol:57,isomorph:[24,25,46,55,62,66,67,77],isprop:5,isquash:12,isquash_sind:12,issac:77,issu:[2,3,24,25,46,52,54,55,58,64,66,71,73],issucc:27,isum:71,iszero:17,ital:[29,53,66,75],italic:[17,75],itarget:17,item:[17,24,25,29,52,54,55,58,60,64,66,67,71,75],iter:[3,5,13,17,25,26,27,28,30,71],iter_add:17,iter_ind:17,iter_invari:17,iter_nat:17,iter_op:17,iter_op_correct:17,iter_rect:17,iter_succ:17,iter_succ_r:17,iter_swap:17,iter_swap_gen:17,ith:46,ito:77,itp:[17,77],its:[2,3,4,5,6,9,10,11,12,13,14,17,24,25,27,28,29,30,31,32,34,35,36,37,38,42,43,44,46,51,52,53,54,55,57,58,59,60,62,63,64,66,67,71,72,73,74,75,77],itself:[2,3,8,9,11,12,13,14,17,30,34,39,40,41,42,43,44,51,53,54,55,57,58,60,63,64,67,71],itzhaki:17,iunit:71,izr:[5,17,71],izr_neq:17,izr_pos_xi:17,izr_pos_xo:17,j:[5,6,8,14,17,24,25,26,34,36,39,43,51,54,57,64,72,77],jablonka:17,jacek:[17,24],jacob:17,jacqu:17,jai:17,jaim:17,jame:17,jan:[17,24,77],januari:[17,24,77],jason:17,jasongross:17,jasper:17,javadoc:75,jean:[2,17,24,77],jedit:17,jef:53,jerri:17,jesper:[17,77],jesu:17,jfehrl:52,jim:17,jm:24,jmeq:[17,67],jmeq_eq_dep:17,joachim:17,job:[8,52,53,54,57],johann:17,john:[5,77],join:[5,24],joint:24,jonathan:17,jone:77,jose:17,jouannaud:77,jourdan:17,journal:77,jouvelot:17,jp:17,jr:17,json:[2,17,51,53,59],juan:17,judg:54,judgement:24,judgment:[26,35,59,77],juli:[17,24],julien:[17,72],julin:17,jump:[8,17,52,57],june:[17,24],jung:17,jurgensen:17,jussieu:17,just:[2,3,4,8,9,11,13,17,24,28,31,34,35,37,41,42,46,51,52,53,55,57,58,59,60,62,64,66,67,71,75],justif:27,justifi:[17,27],jut:24,k1:57,k2:57,k:[2,3,6,14,17,24,26,34,42,54,57,67,72,77],k_1:34,k_i:34,k_j:34,k_n:34,kaiser:17,kaliszyk:17,kalla:17,kamil:17,karl:17,karolin:17,karolina:17,karpiel:17,kartik:17,katakana:29,kate:17,kayla:17,kazuhiko:17,keep:[2,12,14,17,24,33,34,36,42,46,52,53,55,57,64,67],keeper:17,keepsingleton:[2,17],kei:[17,25,41,42,55,57,59,64,66,71],keller:17,kenji:17,kent:77,kept:[14,17,24,36,53,67,75],kernel:[8,9,10,12,24,25,27,29,32,33,36,37,38,41,45,46,53,55,58,59,64,66],ketonen:24,keyboard:[52,59],keystrok:52,keyword:[17,24,25,28,29,32,37,40,46,55,57,64,71,75],khalid:17,khanh:17,kil:17,kill:17,kind:[2,8,10,11,17,25,27,29,34,42,46,53,55,57,59,67,72],kit:17,klausner:17,kleen:[24,60],kloo:17,knaster:24,know:[2,8,17,24,27,32,34,42,46,52,53,54,55,57,59,60,62,64,67,71],knowledg:[17,25,71],known:[2,8,10,12,13,17,24,27,30,33,34,39,41,44,51,55,57,66,71],knownfil:53,knowntarget:53,ko:53,konstantino:17,kosogorov:17,krebber:17,krivin:[17,64],kuefner:17,kunz:17,kuper:17,kw:[0,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],kwend:[0,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],kyoto:24,l0:[46,54,64],l1:[42,54],l1_tactic:54,l2:[42,54],l2_tactic:54,l2r:17,l3_tactic:[54,66],l:[0,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],l_inj:17,l_r_neq:17,la:[13,17,24,52,55,77],lab:24,label:[2,8,14,17,29,54,59],lablgtk2:17,lablgtk3:17,laboratori:24,lack:[17,53,54,57],lafont:[17,77],lam:[26,34],lambda:[2,3,10,11,17,31,52,55,64,67,71,77],lambo:24,lampropoulo:17,land:[5,17,59,71],land_comm:59,land_even_even:17,land_even_l:17,land_even_odd:17,land_even_r:17,land_le_l:17,land_le_r:17,land_odd_even:17,land_odd_l:17,land_odd_odd:17,land_odd_r:17,land_on:59,landau:24,landmark:17,lang:77,langl:17,langston:17,languag:[3,9,11,14,26,29,36,37,39,40,41,46,53,54,63,64,65,66,74,75,77],lannion:24,laport:17,lappli:58,lar:17,larchei:17,larg:[11,14,17,25,26,29,34,35,39,52,53,54,57,61,64,66,67,71,75],larger:[2,13,14,17,25,51,52,57,60,71,75],largest:[57,71],larri:[17,24],lass:[17,77],lasson:17,last:[4,5,9,17,24,32,34,35,37,38,42,46,51,52,53,54,55,57,58,59,60,64,65,66,67,71,72],last_ind_list:57,last_last:17,last_length:17,last_spec:57,last_spec_ind:57,last_spec_rec:57,last_spec_rect:57,last_spec_sind:57,lastadd:57,lastcas:57,lastli:75,lastp:57,lastseq0:57,late:[8,17,24,25,64],later:[11,17,25,31,32,43,44,50,53,55,57,58,66,67,71],latest:[17,25,50],latex:[0,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,54,55,56,57,58,59,60,61,62,63,64,65,66,67,68,69,70,71,72,73,74,76,77],latin1:75,latin:[17,29],latter:[3,11,17,28,34,35,42,51,54,55,57,58,64,66,67,75],lattic:4,launch:[2,13,17,25,52,53],laurenc:[17,57],laurent:[11,17,24],law:[17,24,25],lax:[17,55,60],layer:[10,17,25],layout:17,lazi:[2,8,9,12,17,24,55,64],lazili:[8,17,30,54],lazy_and:17,lazy_goal_match0:17,lazy_impl:17,lazy_or:17,lazymatch:17,lb:13,lbase:17,lceil:5,lcf:[24,55],lcm0:17,lcm:[17,59],lcm_comm:59,ldexp:17,ldexp_spec:17,ldiff:59,ldiff_even_even:17,ldiff_even_l:17,ldiff_even_odd:17,ldiff_even_r:17,ldiff_le_l:17,ldiff_odd_even:17,ldiff_odd_l:17,ldiff_odd_odd:17,ldiff_odd_r:17,ldot:[3,7,34],ldshiftexp:27,le0:42,le:[3,5,13,14,17,24,27,42,46,52,55,57,64,67,77],le_:27,le_add_l:17,le_class:42,le_div2:17,le_div2_diag_l:17,le_epsilon:17,le_eqb:13,le_gt_dec:[2,57],le_ind:[27,46,67],le_ipr:17,le_lt_dec:[2,17,24],le_lt_tran:43,le_m_n:57,le_minu:[17,72],le_n:[27,57,67],le_n_m:57,le_n_p:57,le_not_lt:17,le_plus_r:17,le_rec:67,le_rect:67,le_sind:[27,46,67],le_tran:58,lead:[2,10,14,17,24,26,29,34,39,57,58,60,64,71,74,75],leaf:[34,67],leak:17,learn:[2,17,25,54,72],least:[2,3,12,13,17,25,28,29,30,34,41,46,52,53,57,58,64,66,67,71,72,74,75],leav:[12,13,17,32,35,52,54,57,58,59,60,64,66,67],leb:[5,9,17,27,57,59],leb_implb:17,lectur:77,led:[17,24],ledinot:24,lee:[17,77],lef:46,lefanu:17,left:[0,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,68,69,70,71,72,73,74,75,76,77],lefta:71,leftarrow_:11,leftmost:[17,34,41,58],legaci:[2,3,5,6,9,11,14,17,27,29,34,36,40,42,43,51,54,55,57,58,59,60,64,66,71,72],legacy_attr:[9,14,29,35,40],legal:[17,31,34],legibl:57,legitim:24,lego:24,leibniz:[3,5,7,11,13,17,24,25,27,35,40,57,58,67],leivent:17,lel:59,lel_refl:59,lele_eq:42,leminv:67,lemm:24,lemma:[3,5,11,13,14,17,24,25,32,34,35,36,38,42,44,46,54,57,58,59,60,62,64,67,72],lemmata:17,len:54,lenght:27,length:[0,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],length_app:17,length_combin:17,length_con:17,length_concat:17,length_firstn:17,length_flat_map:17,length_fst_split:17,length_list_pow:17,length_map:17,length_nil:17,length_prod:17,length_rev:17,length_seq:17,length_skipn:17,length_snd_split:17,length_tl:17,length_to_list:17,length_zero_iff_nil:58,lennart:17,lennon:17,leo:[46,67],leonida:17,lepigr:17,leq:[34,42,57],leq_add_sub:57,leqn:57,ler90:[64,77],lerai:17,leroi:[17,24,77],lescuy:17,less:[2,4,8,11,14,17,24,34,46,51,53,54,55,57,59,60,64,71,77],let02:[2,77],let:[0,1,2,3,4,5,6,7,8,9,10,11,12,13,14,15,16,17,18,19,20,21,22,23,25,26,27,28,29,30,31,33,34,35,36,37,38,39,40,41,42,43,44,45,47,48,49,50,51,52,53,55,56,58,59,60,61,62,63,64,65,66,67,68,69,70,71,72,73,74,75,76,77],let_claus:54,letan:17,letin:[0,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],letouzei:[2,17,24,77],lettac:24,letter:[17,24,26,27,29,37,46,51,55,71,75],level:[8,13,14,17,24,25,26,27,31,35,36,37,41,42,46,51,52,53,54,57,59,64,66,67,71,72,73,75],lewycki:17,lex:75,lexer:66,lexic:[2,17,25,51,59,71,75],lexicograph:[7,11,53],lexicographic_exponenti:17,lexicographic_product:17,lfloor:5,lgth:34,lh:[55,57,59],li:17,lia:[17,25,54,55,57,60],lia_ltac1:55,lib:[17,24,51,53,55,59,75],libc:17,librari:[2,5,8,25,29,35,36,40,41,52,54,57,58,64,66,72,75],lic:77,licens:[25,50],licit:25,lid:57,lident:55,life:17,lift:[3,12,14,17],liftn:17,light:[5,17,24,52,66,75],lighter:[8,13],lightweight:17,like:[2,4,8,9,10,11,13,14,17,24,26,27,29,32,34,35,38,39,41,42,43,46,51,52,53,54,55,57,58,59,60,62,64,66,67,71,72,73,75],likewis:[9,17,55],limit:[3,5,8,9,10,13,14,17,24,27,29,35,41,46,51,52,53,54,55,57,58,59,60,63,64,66,71,72],lincon:5,line:[2,8,10,12,14,24,25,29,42,52,53,54,55,57,58,59,64,66,71],lineag:55,linear:[2,3,11,14,17,24,25,46,51,54,55,57,64],linearintuit:24,liner:[17,25],link:[2,16,17,24,27,46,51,53,57,72,75],linker:[2,24],lint:[17,53],linter:[17,51],linux:[17,35,51,52,53,59,64],lionel:17,lip:[24,77],lirmm:77,lisp:24,list0:[55,71],list1:[55,71],list2:34,list2_ind:34,list2_rec:34,list2_rect:34,list2_sind:34,list3:34,list3_ind:34,list3_rec:34,list3_rect:34,list3_sind:34,list:[0,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,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,56,57,58,59,60,61,62,63,64,65,66,67,68,69,70,71,72,73,74,76,77],list_equiv:3,list_ext:17,list_extens:17,list_ind:[14,34,41,44,46,57,67],list_max:17,list_max_app:17,list_max_l:17,list_max_lt:17,list_power_length:17,list_prod_as_flat_map:17,list_rec:[14,34,41,44,46,57,67],list_rect:[14,34,41,44,46,57,67],list_scop:[17,27,64,71],list_sind:[14,34,41,44,46,57,67],list_sum:17,list_sum_app:17,listdec:17,listing_decidable_eq:17,listn:46,listn_ind:46,listn_rec:46,listn_rect:46,listn_sind:46,listnot:[17,54,72],listset:17,listw:34,liter:[2,5,17,29,36,42,54,55,57,71],literatur:[13,34],littl:[8,9,11,14,17,35,57,64],live:[14,17,51,55],live_word:66,ljt:[54,62],ll1:71,ll:[13,17,34,52,53],llm3:24,ln:17,ln_exists1:17,lnc:77,lnot:[17,75],load:[2,3,5,6,7,9,11,17,24,25,27,29,34,35,36,42,43,54,55,57,58,60,64,66,67,71,72,73],loadabl:17,loadfil:59,loadpath:[17,24,51,53,59],local:[2,3,4,5,9,13,17,24,25,26,28,30,31,32,34,41,42,52,55,59,62,64,66,67,75],localis:24,locallysorted_sort:17,locat:[2,17,24,25,35,51,52,53,54,55],lock:[17,25],lockwood:24,log2:[17,59],log2_it:59,log:[17,24,53,54],logarithm:17,logic:[2,3,9,12,13,14,17,24,25,26,28,29,30,34,35,39,51,57,58,59,61,66,67,75,77],logic_typ:[17,27],logical_dir:24,logical_kind:59,logiqu:77,loic:24,loiseleur:[11,24],lone:[17,71],longer:[3,9,17,24,31,34,38,44,52,53,58,66,67,71],longest:[17,29,34,41,42,57,71,75],longrightarrow:[0,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],look:[4,8,9,11,13,14,16,17,25,51,53,54,55,57,58,59,60,66,67,71,72,75],lookup:11,loop:[17,24,25,53,55,58,60,63],loos:[17,60],lopez:17,lor:[17,59],lor_comm:59,lorenzo:77,lose:[34,67,71],loss:[17,57],lost:[17,30,44,57,67],lot:[3,11,17,24,52,55],lotfi:17,lott:17,louis:17,low:[14,17,25],lower:[14,17,25,52,54,55,57,60,64,71],lowercas:[17,29,37,46,52,55],lowest:[37,54],lpar:77,lqa:5,lra:[0,1,2,3,4,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],lri:[17,24,77],ls:[17,51,53],ls_color:51,ls_l:17,lsl:17,lsp:[17,29,74],lsr:17,lt:[3,9,13,17,27,42,57,71,72],lt_1_ipr:17,lt_1_r:67,lt_div2:17,lt_div2_diag_l:17,lt_eq_lt_dec:17,lt_ipr:17,lt_irrefl:[43,58],lt_mult_left:17,lt_n_m:57,lt_not_l:17,lt_tran:[43,57],lt_wf_double_rect:17,lt_wf_rec:[2,24],lt_wf_rect1:17,lt_wf_rect:17,ltac1:[17,25],ltac1_expr_in_env:55,ltac1val:55,ltac2:[25,35,38,52,53,54,59,63,66,71,74],ltac2_as_ipat:55,ltac2_as_nam:55,ltac2_as_or_and_ipat:55,ltac2_atom:55,ltac2_bind:55,ltac2_branch:55,ltac2_by_tact:55,ltac2_claus:55,ltac2_concl_occ:55,ltac2_constr_with_bind:55,ltac2_convers:55,ltac2_delta_reduct:[17,55],ltac2_destruction_arg:55,ltac2_eqn_ipat:55,ltac2_equality_intropattern:55,ltac2_expr0:55,ltac2_expr1:55,ltac2_expr2:55,ltac2_expr3:55,ltac2_expr5:55,ltac2_expr:[55,71],ltac2_for_each_go:55,ltac2_goal_tact:55,ltac2_hypid:55,ltac2_hypident_occ:55,ltac2_in_claus:55,ltac2_induction_claus:55,ltac2_intropattern:55,ltac2_let_claus:55,ltac2_ltac1_plugin:55,ltac2_match_kei:55,ltac2_match_list:55,ltac2_match_pattern:55,ltac2_match_rul:55,ltac2_naming_intropattern:55,ltac2_occ:55,ltac2_occs_num:55,ltac2_or_and_intropattern:55,ltac2_oriented_rewrit:55,ltac2_plugin:55,ltac2_quot:[17,55],ltac2_red_flag:55,ltac2_reduct:55,ltac2_rewrit:55,ltac2_scop:[55,74],ltac2_simple_bind:55,ltac2_simple_intropattern:55,ltac2_simple_intropattern_clos:55,ltac2_typ:55,ltac2_type0:55,ltac2_type1:55,ltac2_type2:55,ltac2_typevar:55,ltac2val:[17,55],ltac:[5,13,24,25,35,38,43,52,53,57,58,59,60,62,63,64,66,67,71,74,77],ltac_expr0:[11,54],ltac_expr1:[54,66],ltac_expr2:[54,66],ltac_expr3:[3,29,54,58,64,66],ltac_expr4:54,ltac_expr:[5,9,11,29,54,55,60,62,64,66,71],ltac_production_item:71,ltacprof:17,ltb:[5,17,27,59],ltnv:57,luca:17,lui:77,lukasz:17,lumsdain:17,luna:24,luo:24,luttik:77,lv97:[3,77],lv:[17,51],lvar:7,lw11:[17,77],lxor:[17,59],lxor_comm:59,lyng:17,lyon:[24,77],lysxia:17,m0:[31,42,67],m150:58,m151:58,m1:[17,35],m2:[17,35],m:[0,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],ma:77,mac:[53,60],maccagnoni:17,machin:[10,17,24,25,27,32,36,51,54,55,64],machineri:[3,17,57],maco:[17,51,52],macro:[17,24,46,66,75],made:[2,3,14,17,24,29,34,35,38,41,46,51,53,54,55,57,58,64,66,71,72,75],magic:[2,17,24,55,59],mahboubi:[11,17,42,57,77],mai:[2,3,4,5,8,9,10,12,13,14,15,17,24,25,26,27,28,29,31,32,33,34,35,37,38,40,41,42,43,44,46,50,51,52,53,54,55,57,58,59,60,62,64,66,67,71,72,73,74,75,77],mail:17,maillard:17,main:[2,8,9,11,13,17,25,27,29,34,40,41,52,53,54,55,57,60,64,71],mainli:[14,60,75],maintain:[9,13,17,39,46,51,53,57,58,71],maintaint:17,mainten:[17,25,58,63],major:[15,17,24,26,42,51,53,55,73,74],makariu:17,makarov:[5,17],make:[2,3,4,5,8,9,10,11,12,13,14,17,24,25,26,27,28,29,30,32,33,34,35,37,38,39,41,42,43,44,45,46,51,52,53,55,57,58,59,60,62,64,66,67,71,75,77],make_a_le_b:14,make_b_lt_c:14,make_change_arg:17,makecmdgo:53,makefil:[17,51,52,53],malecha:17,malici:[17,51],maman:17,man:[25,51],manag:[3,13,17,24,25,32,38,51,53,57,59,60,62,73],mandatori:[2,8,17,32,57,66,71],mangin:17,mangl:[17,51,58,66],mani:[3,11,13,14,17,24,25,27,29,33,34,35,39,42,51,52,53,54,55,57,58,60,64,66,71,73],manifestli:35,manipul:[3,9,10,17,24,25,34,37,39,55,57,63,77],manna:24,manner:[10,24,51],manouri:24,mantissa:27,manual:[2,11,24,25,29,50,52,53,57,60,66,67,71],map2_ext:17,map:[2,3,5,13,17,24,25,26,27,34,35,36,39,41,44,51,53,57,58,59,60,71,72,75],map_append:17,map_const:17,map_eq_app:17,map_eq_con:17,map_ext:17,map_ext_foral:17,map_ext_in:17,map_id:17,map_last:17,map_length:17,map_map:17,map_morph:3,map_repeat:17,map_rev:17,map_shiftin:17,mapl:24,maplemod:24,mapsto:11,marc:17,march:[17,24,77],marech:17,marel:17,margin:[17,57],mari:17,mario:17,mark:[2,12,17,24,31,35,37,38,41,44,51,52,53,54,55,57,59,60,64,66,71],marker:[17,59],marshal:17,marti:17,martin:[17,24,27,34,77],martinez:17,mask:[2,35],massiv:35,master:[8,17,52,53,71,77],master_kei:57,match:[0,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,32,33,35,36,38,39,41,42,43,44,45,47,48,49,50,51,52,53,56,58,59,60,61,62,63,64,65,66,67,68,69,70,71,72,73,74,75,76,77],match_failur:[17,57],match_hyp:54,match_kei:54,match_pattern:54,matches_go:17,matej:17,materi:[17,24,25,50,57],math:[17,75,77],mathbb:[5,7,17],mathcal:[0,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],mathcomp:17,mathemat:[5,17,24,25,29,34,37,51,52,57,64,66,75,77],mathematica:24,mathematician:17,mathematiqu:77,mathieu:77,mathit:[5,26,34],mathrm:[0,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],mathsf:[0,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],mathtt:5,matsushita:17,matt:17,matter:[17,37,51,57,64,67],matth:17,matthew:17,matthia:17,matthieu:[3,9,14,17,77],matur:24,mauni:24,max:[14,17,24,39,46,54,59],max_comm:59,max_int:2,max_length:27,maxim:[3,13,17,25,41,51,57,71,77],maximum:[13,17,27,46,60,62,64,66],mayb:64,mayero:24,mbox:[0,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],mcb00:[67,77],mcbride:[67,77],md5:17,md:[17,71],mean:[2,3,5,9,10,11,12,13,14,17,24,25,26,27,28,29,31,32,34,35,38,40,42,43,44,46,51,52,53,54,57,58,59,64,65,66,71],meaning:[17,29,52],meaningless:75,meant:[2,3,14,17,55,59,64],meantim:17,meanwhil:17,measur:[9,17,34,54,72],measure_induct:17,mechan:[2,3,4,9,10,13,17,24,25,29,34,38,41,46,51,52,53,55,59,64,65,66,71,72,77],medium:57,meerten:6,meet:[2,9,71],melquiond:17,mem:[17,53],member:[13,42,55],memo:24,memoir:24,memori:[8,11,17,24,25,29,51,53],memprof:17,menial:57,mental:67,mention:[2,3,14,17,24,26,34,39,44,46,51,54,57,58,60,64,66,71],menu:[17,24,52,66],mere:[2,17,55,57,64,71],merg:[17,44],mergesort:17,merlin:[17,53],mess:17,messag:[3,4,8,11,12,13,14,16,17,24,26,28,29,30,34,35,37,40,41,42,43,44,46,51,52,54,55,57,58,59,60,62,64,66,67,71,74],met:53,meta:[17,24,25,39,53,59],metadata:[53,59],metalanguag:17,metamathemat:[24,77],metaprogram:54,metasyntact:55,metasyntax:17,metatheori:57,metavari:[17,24,25,54,55,62],method:[2,3,5,6,7,9,11,13,17,24,27,29,30,34,36,42,43,53,54,55,57,58,59,60,64,66,72,77],methodolog:[24,57],metric:17,metzger:17,meven:17,micaela:24,michael:17,michel:[17,24],micro:52,micromega:[17,25,61,66],micromega_core_plugin:[5,11,27,29,36,54,55,57,60,66],micromega_plugin:[5,11,27,29,36,54,55,57,60,66],microsoft:17,mid:17,middl:[17,29,54,57,71,75],might:[2,3,5,13,17,46,51,53,55,57,62,64,67,71,72,75],migrat:17,milad:17,mileston:17,miller:17,milner:[24,55,77],mimic:[13,37,57],mimram:17,min:[17,24,59],min_comm:59,mind:52,mingw:17,minic:24,minim:[8,17,24,25,34,51,53,57,67],minimum:17,miniorderedtyp:17,minki:17,minor:[17,51,57,71],minor_heap_s:51,minu:[11,17,27,29,41,72],minus_ind:72,minus_ipr:17,miquel:24,mirai:17,mirror:17,misc:[17,24,52],miscellan:25,mishandl:17,mislead:[17,71],misleadingli:17,mismatch:[17,46,53],misord:17,mispars:60,miss:[5,10,13,17,24,35,43,51,52,55,57,58,62,64,71,75],misspel:[46,59],mistaken:75,mistyp:10,misus:66,mitchel:77,mitig:[17,57,73],mix:[14,17,24,27,42,54,57,71],mixin:42,mixtur:24,mk_field:11,mk_linear:11,mk_rt:11,mk_sfield:11,mk_srt:11,mkmorph:11,mkpow_th:11,mkpredtyp:17,mkr:17,mkrat:37,mkrel:57,mkrmorph:11,ml4:17,ml:[3,5,6,8,9,11,17,24,25,26,27,29,34,36,42,43,46,51,52,53,54,57,58,59,60,63,64,66,72,77],mldep:17,mlg:[53,59],mli:[5,17,53],mlihtml:17,mllib:[17,53],mlpack:[17,53],mn:17,mod1:[35,51],mod2:[34,35],mod:[0,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],mod_abs_r_mod:17,mod_diveq_iff:17,mod_id_iff:17,mod_mod_abs_r:17,mod_mod_divid:17,mod_mod_opp_r:17,mod_opp_mod_opp:17,mod_opp_r_mod:17,mod_pow_l:17,mod_smal:17,mod_zmod:17,moda:[0,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],modal:17,mode:[9,13,14,17,24,25,29,30,32,34,38,41,46,51,54,58,59,60,65,75],model:[11,17,24,57,77],modern:54,modif:[2,4,11,17,36,41,58,71],modifi:[3,4,8,11,13,14,17,24,25,29,36,38,41,51,52,54,55,57,58,64,66,67,71],modimp:[0,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],modnam:57,modtyp:[0,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],modu:58,modul:[2,3,5,7,9,10,11,13,17,24,25,27,28,29,32,33,36,37,38,40,41,42,44,51,52,54,55,57,58,59,60,64,66,67,71,72,75],modular:[2,17,24],module_bind:35,module_expr_atom:35,module_expr_inl:35,module_prefix:53,module_typ:35,module_type_inl:35,modulenam:75,modulo:[2,4,5,11,17,24,27,34,54,57,58,59,71],modulu:17,moh86:[24,77],mohr:[24,27,77],mohrin:24,moin:17,moment:[17,26,52,53,54],mon_car:14,mon_op:14,mon_unit:14,monad:[14,17,55],monat:[17,24],monin:[17,24],monoid:[14,55],monoid_op:14,monoids_monoid:14,monolith:[2,17],monom:17,monomi:[5,11],monomorph:[9,17,25,27,29],mononorph:14,monospac:17,monoton:[3,4,17],monotoni:3,montevideo:24,month:17,moor:24,mora:77,moral:34,more:[2,3,4,5,6,8,9,10,11,12,13,14,17,24,25,26,27,28,29,30,31,33,34,35,36,38,40,42,44,46,51,52,53,54,55,57,58,59,60,62,63,64,66,67,71,72,73,74,75],moreov:[3,5,17,28,44,46,51,52,57,62,71],morgan:17,morph0:11,morph1:11,morph_add:11,morph_eq:11,morph_mul:11,morph_opp:11,morph_sub:11,morphism:[4,11,17,25,59,71],morphisms_prop:[3,17],morphisms_rel:17,morri:24,most:[2,3,4,10,12,17,24,27,29,34,38,41,45,46,51,52,53,54,55,57,58,60,63,64,66,67,71,72,73],mostli:[2,3,17,24,52,57,60],mot_to_ot:17,motiv:[11,17,55,57,77],motzkin:17,mous:[24,52],move:[13,17,24,25,43,52,53,55,66,67,71],move_loc:55,movement:[17,58],mset:17,msetavl:17,msetrbt:17,msg:55,msub:35,mt13:[42,77],mt:35,mtac2:63,mtac:55,mto:[0,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],much:[2,11,13,17,25,33,51,53,57,59,63,64,71],mul1g:57,mul:[2,5,17,27,36,52,57,59,71],mul_add_distr_l:6,mul_comm:[11,59],mul_exp:57,mul_reg_l:17,mul_reg_r:17,mul_spec:[27,36],mulder:17,mule:57,mulg1:57,mulgi:57,muln0:57,muln1:57,muln:57,mult1_rev:57,mult:[11,17,24,26,27,57],mult_comm:57,mult_ipr:17,mult_mark:57,mult_n_o:27,mult_n_sm:[27,59],multi1:57,multi1_rev:57,multi2:57,multi3:57,multi:[13,17,25,52,54,55,66,75],multi_goal_match0:17,multi_match0:17,multi_match:17,multibyt:17,multimatch:17,multipl:[2,3,4,9,14,17,24,25,27,29,34,35,40,44,52,58,59,60,64,66,67,71],multipli:[2,27,57],multirul:57,multiset_eq:3,multisuccess:17,mun94:[62,77],munch:17,murthi:24,museum:25,must:[2,3,4,6,7,9,10,11,12,13,14,17,24,25,26,27,29,30,34,35,36,37,39,40,41,44,51,52,53,54,55,57,58,59,60,62,64,66,67,71,72,74,75],mutabl:17,mutat:17,mutual:[9,17,24,25,29,30,32,37,54,55,67,71,72],my:[52,53,57,59],my_:40,my_congr_properti:57,my_def:57,my_eq:57,my_lemma1:57,my_lemma2:57,my_nat:40,my_o:40,my_package_plugin:59,my_scop:17,my_tac:52,my_tauto:54,my_tauto_ex1:54,my_tauto_ex2:54,my_toplevel:53,mybool:41,mybool_scop:41,myclass:37,mycod:53,myconst:24,myconstr:55,mye86:[66,77],myer:[66,77],myfield2:37,myfield:37,myfil:53,myfirst:54,myforal:71,mygeneratedfil:53,mylemma:57,mylet:71,mylib:74,myop:57,mypackag:53,myproj:53,myrecord:37,mytac:[17,55,57],mytauto:54,n0:[2,9,31,46,57,58,67,72],n1:[2,9,34,53,57,72],n2:54,n2bv_gen:17,n2bv_size:17,n2z:17,n:[0,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,68,69,70,71,72,73,74,75,76,77],nO:[0,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],n_1:[11,26],n_2:11,n_gt0:57,n_i:57,n_k:26,n_scope:71,n_sn:27,naddord:17,naiv:57,nake:57,name:[2,3,4,5,6,8,9,10,11,13,14,17,25,26,27,28,29,31,32,34,36,38,39,40,41,42,43,44,46,51,52,53,55,57,58,59,60,64,67,71,72,74,75],name_go:66,nameless:[17,77],nameofthem:52,namespac:[10,14,17,35,42,53,59],naming_intropattern:[58,67],nan:[17,27,71],nanci:24,nanevski:77,nant:17,narasimhan:[24,77],narboux:17,narith:[11,17,27],narithr:[11,17],narrow:[59,67],naryfunct:17,nash:17,nat2z:57,nat:[0,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,28,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],nat_cas:[27,67],nat_case_nodep:67,nat_compar:17,nat_compare_alt:17,nat_double_ind:27,nat_eq:42,nat_eqcl:42,nat_eqti:42,nat_ind:[27,34,58],nat_it:17,nat_l:42,nat_lecl:42,nat_leq_compat:42,nat_leqmx:42,nat_leqti:42,nat_leti:42,nat_of_int:2,nat_op:44,nat_or_id:57,nat_or_var:[5,13,17,54,58,60,67],nat_rec:[27,34,44,67],nat_rec_nodep:67,nat_rect:[2,27,34,59],nat_rect_plu:59,nat_scop:[6,27,31,34,38,46,57,71],nat_setoid:42,nat_sind:[27,34],nati:53,natint:17,nativ:[2,5,10,12,24,25,36,51,55,58,59,64],native_cast_no_check:58,native_comput:[17,25,32,36,51,58],native_compute_profil:64,nativecomput:[17,64],natnod:34,natord:17,natpair:17,natr:24,nattre:34,nattree_ind:34,nattree_rec:34,nattree_rect:34,nattree_sind:34,natur:[2,5,7,9,13,14,17,24,25,26,27,28,29,30,34,35,37,39,40,42,44,46,52,53,57,58,59,62,64,66,71,72],naveen:17,navig:[17,24,52,57,75],nawrocki:17,nbinari:[17,53],ncring:17,ncring_tac:17,nd:77,ndefop:17,ndigit:17,ndist:17,ndoubl:17,ne_:71,nearest:[17,27,54],nearli:73,necess:17,necessari:[3,4,9,13,17,24,29,31,33,37,53,55,57,59,62,64,67,71],necessarili:[4,46,67,72],necessit:24,need:[2,3,5,8,9,10,11,13,14,17,24,25,28,29,31,32,34,35,38,41,42,43,44,46,51,52,53,54,55,57,58,59,60,62,64,66,67,71,73,75,76],needless:60,neg:[5,17,27,29,30,37,64,66,71],neg_infin:27,neg_zero:27,negat:[17,27,54,57,58,60,62,67],negb:[5,13,27,62,71],negp:57,negpp:17,neither:[10,14,17,46,54,55,57,64,67],nelson:62,neq0:57,neq:11,neq_symmetr:59,neqb:13,neqb_implicit:13,nest:[3,9,17,24,25,29,32,35,38,40,54,57,58,59,64,66,71,75],net:17,network:60,never:[2,13,14,17,24,35,41,42,44,51,54,55,57,58,60,64],nevertheless:[2,17],new_goal:17,new_var:17,newcommand:[0,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],newdestruct:[17,24],newer:17,newest:[7,54,55],newinduct:[17,24],newli:[17,60,67],newlin:[17,24,29,53,54,71,75],newman:[17,24],newn:54,next:[3,9,13,17,24,27,29,33,34,42,44,46,51,52,54,55,57,60,64,65,66,67,71],next_down:27,next_up:27,ngan:17,nge0:57,ngt0:57,ni:53,nia:[17,25],nice:[52,57,67,75],nicer:17,nichola:17,nick:17,nickolai:17,nicola:[3,17,77],nicolo:17,niel:17,niesi:77,nijmegen:[17,24],nikishaev:17,nikita:17,nikolao:17,nil2:34,nil3:34,nil:[0,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],nil_spec:17,nilhl:[0,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],niln:46,nilw:34,ninf:27,niqui:17,niso:17,nix:17,nlist:71,nm:57,nmake:17,nmake_gen:17,nmax:17,nmin:17,nminu:17,nnn:[17,71],nnormal:27,nnumber:17,noccur_between:17,noccurn:17,nocor:[17,60],nocycl:53,node:[0,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],nodebug:17,nodup:17,nodup_app:17,nodup_app_remove_l:17,nodup_app_remove_r:17,nodup_concat:17,nodup_filt:17,nodup_iff_forallordpair:17,nodup_incl:17,nodup_incl_nodup:17,nodup_list_decid:17,nodup_map_nodup_forallpair:17,nodup_permutation_bi:17,nodup_rev:17,noedit:66,noi:[17,51],noinit:[17,29,51,66],noinlin:2,nois:53,nomacintegr:17,nomatch:[17,41],non:[2,4,6,8,9,10,13,14,17,24,25,26,27,28,29,30,35,37,40,41,46,51,52,53,57,59,60,62,64,66,72,75],nonassoci:71,nonconst:7,noncrit:17,noncumul:[17,25,29],none:[4,5,13,17,24,27,34,40,42,46,51,54,55,57,66,71],nonempti:60,nonetheless:[2,17,30,32,36,51,66],nonlinear:17,nonneg:60,nonprimit:17,nonproptyp:17,nonrecurs:[17,37,40,67,72],nonreflex:25,nonsimple_intropattern:55,nonstandard:17,nonsymmetr:25,nontermin:[17,29,54,55,71],nontrivi:[11,17,46,51,57],nonuniform:[4,17],nonzero:[3,11,37,54],nor:[10,11,17,26,34,35,46,51,52,53,54,55,57,58,59,64,67,71],norec:51,norm:11,normal:[2,3,4,5,11,17,24,26,27,29,30,31,34,35,41,44,51,52,53,54,55,57,59,64,66,67,71,72,77],normfr_mantissa:27,norp:57,north:77,nosimpl:57,not_1_ipr:17,not_eq_:27,not_eq_sym:27,not_found:[17,24],not_i:34,not_i_i:34,not_ipr:17,not_locked_false_eq_tru:17,not_nodup:17,nota:17,notabl:[10,17,24,37,51,55,57,64,67],notat:[4,5,9,10,11,14,24,25,26,28,29,31,33,34,35,36,37,38,40,41,45,46,51,52,53,57,58,60,64,67,73,74,75,77],notation_declar:71,notconst:11,notcresolut:[17,57],note:[2,3,4,5,7,8,10,11,12,13,14,15,17,24,26,27,28,29,34,35,37,40,41,42,43,46,51,52,53,54,55,57,58,59,60,62,64,66,67,71,72,74,77],notempl:17,notepad:53,noth:[3,17,38,41,51,54,55,57,58,62,64,66,67],notic:[3,4,5,17,26,34,35,38,46,51,52,54,57,58,64,66,71,72,74],notin:[17,26],notin_flat_map_foral:17,notin_remov:17,notion:[5,11,17,24,25,26,27,33,34,46,51,54,55,58,64,71,77],nott:[17,27],notypeclass:[17,58],nouniv:54,nov:24,novel:[17,25],novelti:[17,25],novemb:[17,24,77],novic:[17,57],now:[2,3,4,11,13,14,17,24,26,27,30,34,35,41,42,46,51,52,53,54,55,57,59,60,64,67,71,72,74],np_n:34,npe:11,npeano:17,npo:37,nq:67,nra:[17,25],ns:[0,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],nsatz:[17,25,61],nsatz_comput:17,nsatztact:[7,17],nset:71,nsi:17,nsubn:27,nsucc_doubl:17,ntf:51,nth:[17,27,58],nth_append_l:17,nth_append_r:17,nth_error:17,nth_error_:17,nth_error_app:17,nth_error_con:17,nth_error_cons_0:17,nth_error_cons_succ:17,nth_error_ext:17,nth_error_firstn:17,nth_error_map:17,nth_error_nil:17,nth_error_o:17,nth_error_repeat:17,nth_error_rev:17,nth_error_seq:17,nth_error_skipn:17,nth_ext:17,nth_middl:17,nth_nth_nth_map:17,nth_order:17,nth_order_ext:17,nth_order_hd:17,nth_order_replace_eq:17,nth_order_replace_neq:17,nth_order_tl:17,nth_repeat:17,nth_replace_eq:17,nth_replace_neq:17,ntn:24,nullstellensatz:[5,7,17],num1:24,num2:24,num:[11,17],numarg:24,number:[2,3,4,5,7,8,11,13,14,17,24,25,26,29,30,34,36,37,39,40,41,42,43,44,46,52,53,55,57,58,59,62,64,66,67,72,74,77],number_modifi:71,number_or_str:[29,71],number_string_via:71,numer:[5,11,17,24,27,29,59,71],numgoal:[17,25],nuprl:24,nvar:24,nw:2,ny:77,nz:17,nzdomain:17,nzero:27,nzmulord:17,nzmulorderprop:17,nzprop:17,nzproperti:17,o:[0,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],o_:[27,37],oapp_comp:17,obei:[17,24,37],obfusc:59,obindeapp:17,obj:[2,24,42],object:[2,3,4,8,9,11,13,14,17,24,25,26,28,29,30,31,33,35,37,38,39,40,41,42,44,51,53,55,57,59,64,67,71,72],oblig:[13,17,25,37,57,62,72],observ:[17,34,37,40,54,55,59,66,71],obsolet:[6,17,24,51,58],obstacl:[17,42],obstruct:57,obtain:[2,3,4,5,17,34,36,54,55,57,58,64,67,72,75],obviou:[3,34,57,71],obvious:17,ocaml:[2,11,17,24,25,27,29,32,36,51,53,54,55,63,64,66,71,73,75],ocaml_librari:53,ocamlbuild:17,ocamlc:17,ocamldep:17,ocamldoc:75,ocamlfind:[17,53,59],ocamllib:53,ocamlopt:17,ocamlrunparam:[17,51,66],ocamlwarn:53,ocan_comp:17,ocan_in_comp:17,occ:57,occ_switch:57,occas:17,occasion:[17,24,29,53,66],occs_num:[17,55,58,64],occur:[2,3,4,8,17,24,26,28,30,34,37,38,41,42,44,46,54,55,57,58,59,60,64,66,67,71],occur_between:17,occurn:17,occurr:[2,3,11,14,17,24,25,26,43,44,46,52,54,55,59,60,64,71],octal:17,octob:[24,77],ocurr:58,odd:[0,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,68,69,70,71,72,73,74,75,76,77],odd_:34,odd_alt:17,odd_alt_odd:17,odd_even:[17,67],odd_even_ind:17,odd_ind:[34,67],odd_j:57,odd_odd:17,odd_sind:[34,67],odditi:54,oddn:57,oddt:17,oddt_event_rect:17,of_bit:59,of_constr:55,of_float:36,of_goal:17,of_hex_uint:59,of_int63:27,of_int64:36,of_int:[17,36],of_intro_pattern:17,of_list_to_list_opp:17,of_module_typ:35,of_nat:[17,57],of_num_uint:[29,59,71],of_preterm:17,of_str:55,of_typ:[4,17,28],of_type_inst:[17,34,37],of_uint:[59,71],of_uint_dec:71,off:[2,8,10,12,13,14,17,24,27,29,34,35,37,43,44,46,51,52,53,54,57,59,64,66,67,71],offer:[17,29,46,51,52,54,57,59,71],offici:[17,54],offset:[17,27,53],offsid:17,ofil:53,often:[2,3,10,13,14,17,25,28,43,46,52,53,54,55,57,58,66],ok:[17,29,52,58],okada:17,okj:17,old:[3,11,24,25,51,53,55,58,60,66,67],older:[17,29,51,67],oldest:[4,17],oldf:55,oldroot:17,olift:17,olift_comp:17,oliv:17,olivi:[17,24],omap_comp:17,omapeapp:17,omapebind:17,omega2:17,omega:[17,24],omegalemma:17,omegatact:17,ominu:11,omiss:17,omit:[2,3,8,14,17,27,28,29,30,32,34,37,38,40,41,42,44,45,46,53,54,55,57,58,59,60,66,67,71,75],omnisci:17,onc:[3,8,9,10,11,13,14,17,24,25,27,32,34,41,42,44,46,51,53,55,57,58,59,60,64,66,67,71,72],ondemand:[17,51],one:[2,3,4,5,6,8,9,11,12,13,14,15,17,24,26,27,28,29,30,31,33,34,35,36,37,38,40,42,43,44,46,51,52,53,54,55,57,58,59,60,62,63,64,66,67,71,72,74,75,77],one_goal_match0:17,one_minus_one_is_zero:36,one_pattern:[13,59,60],one_term:[3,5,7,11,13,29,34,54,58,60,62,64,67,71,72],one_term_with_bind:[3,58,64,67,72],one_two_ir:37,one_typ:[29,58,64],ones:[2,3,4,6,8,13,14,17,25,28,34,35,37,44,46,52,53,54,57,58,59,63,66,67,71,75],ones_0:17,ones_succ:17,ongo:[17,63],onli:[2,3,4,5,6,7,8,9,10,11,12,13,14,17,24,25,26,27,28,29,30,31,32,33,34,35,37,38,39,40,41,42,43,44,46,50,51,52,53,54,55,57,58,59,60,62,64,66,67,71,72,73,74,75],onlin:[27,73],onto:[17,71],oop:17,op1:[57,58],op2:58,op:[5,42,44,53,57,66,71],opac:[17,59,64],opam:[17,25,27,73],opam_packag:53,opaqu:[3,6,8,9,14,17,24,25,31,32,35,38,51,57,59,60,64,66,67,71,75],opcod:17,open:[3,5,6,11,13,17,25,27,35,36,38,42,50,52,54,55,57,59,60,64,66],open_bind:[6,28,58,64],open_constr:[17,55,71],open_constr_flag:17,open_constr_with_bind:17,openbsd:17,opencont:[25,50],openpub:[25,50],oper:[3,5,9,10,11,14,17,24,25,27,32,34,36,51,52,54,55,57,60,64,66,67,71],operand:[17,27,64],operation:36,operators_properti:17,opl:5,oplt:5,oplu:11,opn:58,opp:[17,27],oppen:62,opportun:17,oppos:[17,57],opposit:[17,31,32,46,58,64],opt:[17,24,53,55,71],optim:[5,9,17,24,25,36,58,64,66,77],optimis:24,optimize_heap:[17,66],option:[5,8,9,10,11,13,14,16,24,25,26,27,34,35,38,40,42,44,46,50,52,53,54,55,57,58,59,60,62,64,67,71,74],option_eqb:13,option_eqb_obligation_1:13,option_eqb_obligation_2:13,option_eqb_obligation_3:13,option_ind:[27,34,58],option_rec:[27,34,58],option_rect:[27,34,58],option_sind:[27,34,58],oq:77,or_and_intropattern:58,or_assoc:59,or_ind:[34,40],or_introl:[27,34,40,46,58,67],or_intror:[27,34,40,46,58,67],or_sind:[34,40],oracl:5,orang:52,orb:[2,27,57,62],orb_comm:59,orb_negb_l:17,ord:[13,57],ord_ind:57,ord_rec:57,ord_rect:57,ord_sind:57,order:[2,3,4,6,7,8,9,11,12,13,14,15,17,24,25,26,27,29,30,32,34,35,37,40,42,43,46,51,52,53,54,55,57,60,61,62,64,66,67,71,72,75,77],ordered_set_lang:53,ordered_typ:[17,60],orderedgrammar:71,orderedtyp:[17,60],orderedtypeex:17,orderg1:57,orderg:57,orderg_dvd:57,ordersex:17,orderstac:17,ordinari:[3,17,26,37,39,71],org:[25,50,64,75,77],organ:[17,24,25,53,54,57],organis:24,orient:[17,24,25,51,54,55,57,60,64],oriented_rewrit:[55,64],origin:[2,3,4,9,11,17,24,29,31,34,38,43,44,46,53,57,58,62,64,66,67,71],orp:57,orphan:53,orphan_foo_bar:53,orpp:17,orsai:[17,24],orthogon:57,os:[17,53],oscar:17,ot:60,other:[2,3,4,5,8,9,10,11,12,13,14,24,25,26,27,28,29,30,31,32,33,34,35,36,37,38,41,42,43,51,52,53,54,55,57,58,59,60,62,63,64,67,71,72,76],other_const:42,otherwis:[2,3,9,13,14,17,28,29,34,41,42,44,46,51,52,53,54,55,57,58,59,62,64,66,67,71,73],otim:11,our:[4,5,7,11,17,24,34,35,54],ouri:77,ourselv:[14,34],out:[8,17,24,29,42,52,53,54,57,58,59,60,66,71,75],outcom:[17,51,53,54,67],outdat:17,outer:[14,17,46,66],outermost:67,outperform:17,output:[2,3,4,11,14,17,24,33,42,51,52,53,54,59,60,64,66,71,75],output_valu:17,outputst:17,outsid:[3,5,9,11,12,13,14,17,28,29,35,38,40,41,42,43,53,54,59,60,66,71],ouvert:77,over:[2,3,11,14,17,24,25,26,27,28,30,32,34,37,38,39,40,41,42,44,46,52,53,54,58,59,60,61,62,64,66,67],overal:[51,54,64,75],overflow:[2,17,59,66,71],overhaul:17,overhead:[17,53,64],overlap:[5,17,42,46,53,57,59,66],overli:17,overlin:[0,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],overload:[17,24,25,71],overrid:[2,14,17,37,51,53,57,66,67,71],overridden:[17,27,54,57,71,75],overriden:17,overview:[17,25,71],overwrit:[52,64,66],overwritten:75,ovl:[0,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],ow:55,own:[5,10,17,24,25,35,42,44,54,57,59,60,62,66,67,75],owr:77,p0:[9,31,67,72],p1:[13,17,37,57,67],p2:[37,57,67],p2q:57,p:[0,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],p_0:5,p_1:[5,7,34,35],p_2:[5,35],p_:[7,34],p_i:[7,34],p_j:[5,34],p_l:34,p_m:34,p_p:34,p_r:[34,35],p_rmin:17,p_u:34,p_unit:54,p_xy:57,pa:57,pab:57,pablo:17,pack:[3,42,53],packag:[17,24,25,35,42,51,52,59,67,73,75],packtyp:14,pad:57,page:[17,25,27,51,52,71,75],pain:57,pair:[0,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],pair_eq:42,pair_eqcl:42,pair_eqti:42,pair_l:42,pair_lecl:42,pair_leq_compat:42,pair_leqmx:42,pair_leqti:42,pair_leti:42,pairusualdecidabletypeful:17,pairwis:57,palaiseau:17,palat:[17,55],pale:66,palmskog:17,pane:52,panel:[8,17,52,66],panic:55,paolo:17,paper:[13,24,42,54,57,72,77],par95:[9,77],par:[8,17,52,54],paradigm:24,paradox:[34,77],paragraph:[11,27,35,40,57,75],paral:17,parallel:[17,24,25,38,51,52,53,54,57,76],param:17,param_1:17,param_n:17,paramet:[3,4,5,7,8,13,14,17,24,25,28,29,34,37,40,41,43,44,53,54,55,58,59,60,64,66,67,71,72],parameter:[3,5,11,14,17,24,25,28,37,40,54],parametr:[17,24,25,34,40,64],parent:[9,17,24,77],parenthes:[2,3,8,17,24,28,29,35,37,46,54,55,57,58,67,71],parenthesi:[17,57,66],pari:[17,77],parimala:17,parith:[17,27],pariti:17,parm:71,parrai:[17,36],pars:[9,17,25,27,29,41,42,46,51,54,57,59,60,74,75],parse_entri:17,parser:[14,17,24,29,53,71],parsimoni:57,part:[2,3,10,11,13,15,17,24,25,27,29,34,35,37,46,51,52,53,54,55,57,58,66,67,71,72,73,74],parti:[17,51,52,53,59,75],partial:[3,13,17,24,34,35,37,44,51,53,54,57,59,62,66,71,72],particip:[17,57],particular:[2,3,6,9,10,12,13,17,29,30,31,32,33,34,37,38,40,42,52,53,54,55,57,59,60,64,66,71,75],particularli:[17,25,42,51,53,64,71],partit:17,partition_as_filt:17,partli:[17,57],partner:17,pascal:17,pass:[3,5,8,10,12,17,24,37,38,42,51,52,53,54,55,57,60,64,66,67,71,75],past:[2,17,52,64],pat1:17,pat:[17,55],patch:17,patenaud:17,path:[2,4,5,17,24,25,27,35,51,52,54,60],pathnam:[51,53],patholog:2,patn:17,patrick:[11,24],pattern0:[28,40],pattern10:40,pattern1:40,pattern:[2,9,13,17,24,25,27,28,30,32,34,40,41,42,45,60,64,67,72,77],pattern_occ:[58,64],paul:17,paulin:[17,24,27,34,77],paulson:24,pautomata:24,pave:17,payload:27,pb:57,pc:11,pcan_in_comp:17,pcan_in_inj:17,pcm:17,pcompar:17,pcoq:24,pdf:[17,29,77],pe:11,peadd:[5,11],peak:[17,53,66],peano:[17,24,25,34,57,60,71],peano_dec:24,peanonat:[6,17,58,59],pec:[5,11],pedant:59,peeval:11,pemul:[5,11],pen:57,pennsylvania:[17,77],peopl:17,peopp:11,pepow:11,per:[2,3,11,17,24,52,53,57,59,71],per_symmetr:59,percentag:54,perf:[17,64],perfectli:2,perfetto:51,perform:[2,3,5,7,8,11,13,17,24,25,26,34,41,42,46,51,54,55,57,60,62,64,66,67,71,72],perfum:17,perhap:[52,53,58],period:[17,24,29,52,54,60,66,74],perm:54,perm_append:54,perm_aux:54,perm_con:54,perm_ind:54,perm_refl:54,perm_sind:54,perm_tran:54,permiss:[17,53],permit:[9,17,24,25,34,37,38,53,54,55,58,60,64,66,67,71],permtat:17,permut:[3,17,25,55,57],permutation_app:17,permutation_app_inv_m:17,permutation_app_middl:17,permutation_app_rot:17,permutation_app_swap_app:17,permutation_con:17,permutation_count_occ:17,permutation_elt:17,permutation_elt_map_inv:17,permutation_exist:17,permutation_flat_map:17,permutation_foral:17,permutation_forall2:17,permutation_imag:17,permutation_incl_cons_inv_r:17,permutation_ind_transp:17,permutation_list_max:17,permutation_list_sum:17,permutation_map_inv:17,permutation_map_same_l:17,permutation_middle2:17,permutation_morph_transp:17,permutation_permutation_transp:17,permutation_pigeonhol:17,permutation_pigeonhole_rel:17,permutation_refl:17,permutation_repeat:17,permutation_transp:17,permutation_transp_con:17,permutation_transp_equiv:17,permutation_transp_sym:17,permutation_vs_cons_cons_inv:17,permutation_vs_cons_inv:17,permutation_vs_elt_inv:17,permutsetoid:17,perri:17,persist:[9,17,24,29,35,36,38,64,77],person:[24,64],perspect:[24,77],pertain:54,pervas:17,pesub:11,peter:[17,24],peterson:17,pex:[5,11],pexpr:11,peyton:77,pf_type_of:17,pf_unsafe_type_of:17,pfen:[17,24,77],pff:8,pfst:14,pg:[17,66],pgdn:17,pgivesbound:8,pgup:17,phantom:42,phantom_ind:42,phantom_rec:42,phantom_rect:42,phantom_sind:42,phase:[17,24,52,54,55,57,64,72],phd:[24,77],phi:17,philosoph:11,phoni:[17,53],phrase:[25,71],physic:[17,24,35,51,53,59,75],physical_dir:24,phyumn5ooqtymh4h6i0nsskchnaysu:51,pi:[13,17,52],pi_:28,pichardi:[72,77],pick:[17,42,51,52,53,57,58,66,67],pictur:17,pide:17,pident:14,piec:[11,42,43,53,55,57],piecewis:17,pierc:17,pierr:[2,17,24,77],pile:57,pinf:27,pinj:11,pink:52,pinot:17,pinpoint:57,pioneer:24,pipe:17,pise:24,pit:17,pittsburgh:77,pivot:5,pk:[14,57],pkg:[53,59,75],pl:55,place:[2,3,17,32,40,43,51,53,57,58,59,64,66,67,71,75],placehold:[17,43,44,51,57,58,66,71],plai:[2,17,26,42,64,66],plain:[9,17,35,57,75],plainli:55,plan:[10,17,25,53,55,72],plane:[17,24,25],platform:[17,24,36,51,53,54,72],pleas:[17,24,44,53,54,55,62,66,67,72,77],plu:[0,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],plug:59,plugin:[2,5,11,12,17,24,25,29,33,35,53,54,55,59,63,66,71,72],plugin_tutori:[17,63,74],plumb:67,plural:[17,28,38],plus0l:60,plus0r:60,plus1:71,plus_assoc_reverse_stt:59,plus_equ:[57,72],plus_fct:41,plus_ind:[57,72],plus_ipr:17,plus_n_o:[27,59],plus_n_sm:[27,59],plus_o_n:59,plus_rec:[57,72],plus_rect:[57,72],plus_sn_m:59,plussl:60,plussr:60,pm89:[24,77],pm93a:[31,77],pm93b:[24,77],pm:57,pmult:17,pmult_comm:17,pn:[13,17,57],pnormal:27,po:[17,24,59,71],point:[2,3,11,13,17,24,25,26,27,32,34,35,36,39,51,52,53,54,55,57,66,71],pointer:[24,26],pointless:57,pointwis:3,pointwise_rel:3,pol:11,polici:[17,57,74],pollack:24,polylist:24,polymorph:[2,3,13,17,24,25,26,27,29,30,31,32,33,37,39,40,41,44,46,51,59,66,67,71],polynom:11,polynomi:[5,7,17,24,25,61],ponen:58,pool:[17,62],poor:17,poorli:[43,54],pop:[57,71],popl:77,popul:29,port:[3,17,24,55,72],portegi:17,portion:[17,57],pos_neg_int63:71,pos_sub:17,pose:[5,17,24,34,54,55,57,58,67],posit:[3,4,5,7,9,10,11,14,17,24,25,27,30,36,37,39,41,44,46,51,52,54,55,57,58,59,64,66,67,71],position:[2,58],positive_as_ot:17,positive_scop:[27,71],positiveint:55,positivstellensatz:[17,25],posreal:17,possibl:[2,3,4,5,8,9,11,13,14,17,24,27,28,31,34,35,37,41,42,43,44,46,51,52,53,54,55,57,58,59,60,64,66,67,71,73,74,75],post:[17,24,53,57],postfix:[17,57,71],postpon:[17,58,66],postprocess:11,postscript:75,postul:28,potenti:[9,13,25,42,46,52,54,55,57,67,71],pottier:[7,17,24,57],poulin:17,poulsen:17,pow:[5,17,27,59],pow_div_l:59,pow_inv:17,pow_ipr:17,pow_lower_bound:17,pow_n:11,pow_po:[17,71],power:[4,5,11,17,24,27,54,57,67,71,72],power_theori:11,powerrz:17,powerrz_inv:17,powerrz_mult:17,powerrz_neg:17,powerset:34,pp:[17,53],ppair:14,pphi_dev:11,pphi_dev_ok:11,pplu:10,pplus_rewrit:10,ppm89:[24,77],pprod:14,pqequiv:57,pr1:14,pr2:14,pr:17,pr_numgoal:54,pr_p:57,practic:[2,3,5,17,24,25,32,34,39,42,53,55,57,58,64,66,71,74,77],pre:[2,17,25,53,60],preambl:75,preced:[17,25,27,29,46,54,57,58,60,66,75],preceed:64,precis:[4,8,13,17,24,26,29,31,33,34,35,37,39,46,51,57,64,71],precisionnotzero:8,precompil:[17,25,51,64],precondit:58,pred:[9,17,27,54,57,59,60,64],pred_add:64,pred_class:17,pred_doubl:17,pred_n:17,pred_oapp:17,pred_sn:27,pred_sort:17,predecessor:27,predefin:[11,24,25,51,52,66],predic:[3,9,17,24,25,26,27,30,34,40,42,54,60,64,77],predict:[14,17,54,64],predtyp:17,preexist:17,prefac:60,prefer:[7,17,25,34,51,53,57,58,59,62,66,71],preferenti:71,prefix:[2,3,9,11,14,17,24,27,28,34,35,38,40,41,42,44,51,52,54,57,58,59,64,66,67,71,75],preformat:75,preimag:17,preliminari:11,prelud:[2,17,25,29,51,59,66],premis:[17,24,28,35,57,60,66],prenex:57,preomega:17,preorder:[13,57,59],preorder_reflex:[13,59],preorder_transit:13,prepar:[17,24],prepend:[51,53,66],preproccess:17,preprocess:[11,17],preprocessor:[11,24],prerequisit:[17,53],presburg:24,prescrib:[17,57],presenc:[8,17,24,34,44,46,57,64,72],present:[2,3,6,9,11,13,15,17,24,25,26,29,30,32,33,34,37,41,42,44,45,46,50,53,54,55,57,58,59,60,61,63,64,65,66,67,71,73,74,75,76],preserv:[2,5,14,17,24,25,29,30,34,42,55,57,64,67,71],press:[52,77],pressur:60,presum:[17,71],presuppos:[5,75],preterm:[9,17,55],pretti:[17,24,25,27,51,53,57,59,71],pretyp:[17,51,55],prevail:34,prevent:[13,17,29,34,41,42,51,53,54,57,64,71],preview:[2,52],previou:[2,3,4,8,9,11,13,15,17,24,27,29,31,34,37,40,41,42,45,46,51,52,54,55,57,59,60,62,64,66,67,71,74],previous:[2,13,17,28,34,38,52,54,57,59,71],prf_equiv:42,prim2sf:[27,36],prim:[17,71],primari:[52,54],primarili:[32,34,58,66],prime:[3,17,29,34,57],prime_decomp:57,prime_i:57,primfloat:[17,27,36,59,71],primfloatnot:17,primint63:[36,59,71],primit:[2,10,12,13,14,17,24,25,30,33,34,41,46,54,55,57,64,67],primstr:[27,36,71],primstringaxiom:27,princ:17,princeton:17,princip:[17,24,34,57,72,77],principia:24,principl:[2,5,17,24,25,27,30,34,37,51,57,58,63,64,71,77],print:[2,5,6,8,11,12,13,17,24,25,27,29,31,34,35,36,38,39,41,42,51,52,53,57,58,60,62,64,66,67,74],print_list:55,printabl:71,printconf:59,printer:[17,24,29,46,57,59,71],printf:17,prior:[17,51,54],prioriti:[13,17,37,46,52,57,59,66,71],prisqu:17,privat:[13,14,17,25,29,30,34,37],private_:[17,59],probabl:[2,17,32,44,51,54,57,58,59,75],problem:[2,4,7,9,13,17,24,29,34,42,44,46,51,52,53,54,58,62,66,67],problemat:[40,55],proc:77,proce:[3,11,13,52,57,71],procedur:[3,4,11,17,24,25,54,57,60,62,64,77],proceed:[58,77],process:[9,11,14,17,24,25,26,30,32,35,41,42,51,52,53,55,57,58,59,60,64,66,67,75,76],processor:[17,27,36],prod:[2,17,26,27,34,46,62,67],prod_:57,prod_appvect:17,prod_curri:17,prod_curry_uncurri:17,prod_eqb:13,prod_eqb_obligation_1:13,prod_f_r0:17,prod_f_so:17,prod_ind:[27,34],prod_length:17,prod_monoid:14,prod_of_sigt:17,prod_rec:[27,34],prod_rect:[27,34],prod_sigt_prod:17,prod_sind:[27,34],prod_uncurri:17,prod_uncurry_curri:17,prodimp:26,prodt_curri:17,prodt_uncurri:17,produc:[2,5,7,8,9,11,13,14,17,24,25,29,32,34,36,38,40,41,44,52,53,54,55,57,64,66,71,72,73,74,75],product:[2,3,5,10,11,13,14,17,24,26,27,28,34,36,39,40,46,54,55,57,59,60,64,66,67,71],prof:[17,53],profil:[5,17,25,53,59,64],program:[0,1,3,4,5,7,8,10,11,12,13,14,15,16,17,18,19,20,21,22,23,24,25,26,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,56,57,58,59,61,62,63,64,65,66,67,68,69,70,71,72,73,74,75,76,77],program_branch_0:[9,13],program_branch_1:[9,13],program_branch_2:13,program_scop:17,program_simpl:9,programm:[3,24,25,65],programmat:13,progress:[3,17,24,25,51,52,55,60,66,77],progress_evar:17,proj1:[27,66],proj1_sig:[17,46,57],proj2:27,proj:[17,24,54],project:[2,3,9,10,12,13,14,15,17,24,25,27,29,30,34,40,41,42,51,52,54,55,57,59,60,64,72,73,74,76],projections2:27,projs1:24,projs2:24,projt1:[17,27],projt2:27,projt3_eq:17,prolog:[17,24,60],prompt:[17,24,52,54,59],prone:[54,57],proof:[2,3,6,7,9,11,13,17,24,26,27,29,30,33,34,36,37,38,39,40,42,43,44,51,52,53,55,59,61,62,64,67,72,73,74,75,76,77],proof_admit:17,proof_irrelev:34,proofgener:53,prooftre:[17,59,66],proofview:55,prop:[0,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,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],propag:[3,11,17,41],propbinop:5,proper:[3,9,17,24,54,55,59,67],proper_prf:17,properli:[2,8,9,10,17,29,52,53,57,59,66],properti:[3,4,6,9,11,12,13,17,24,25,26,27,30,31,32,34,38,39,42,45,46,57,58,67,72,77],propextension:17,propop:5,proport:64,propos:[17,24,34,54],proposit:[2,3,5,10,17,24,25,26,28,29,30,31,32,33,34,39,40,51,57,58,62,64,66,67,77],propositionnel:77,propr:24,propuop:5,prose:17,protect:[11,17,30,57],protocol:[17,77],protonmail:17,prototyp:[9,17,24],provabl:[5,11,17,34,39,57,58,66],prove:[3,5,7,8,9,11,17,24,25,27,30,32,34,35,42,43,57,58,60,62,64,72,77],proven:[11,17,52,58,64,66,67],prover:[4,5,15,17,24,26,29,31,33,52,55,59,65,73,75,76],provid:[2,5,6,7,8,9,10,11,12,13,14,15,16,17,24,25,26,27,29,30,32,33,34,35,36,37,41,42,43,44,51,52,53,54,55,57,58,59,60,62,63,64,65,66,67,71,72,73,74,75],provis:62,prune:[38,57],ps:75,psatz:[17,25],psatzadd:5,psatzc:5,psatzin:5,psatzmul:5,pseudo:[17,57,60],psnd:14,pstring:[27,36],psubn:27,publi:77,public_nam:53,publicli:17,publish:[24,53,77],puech:17,puf:77,pull:[17,55],pun:[17,55],punctuat:[71,75],pure:[3,7,11,17,55,57,64,71,72,75],purifi:17,purpos:[12,14,17,24,27,34,35,42,51,52,54,55,57,59,64,66,67,71],push:[2,17,57,71],put:[3,5,13,14,17,34,35,43,51,53,54,57,58,59,60,66,67,71,72,75],putnam:24,puydt:17,puzzlement:24,pv:[9,77],pwd:[2,14,59],px:[11,24,57],py:17,python2:17,python3:17,python:[17,53],pzero:27,q1:[5,10,13,46,57],q2:[5,10,57],q2p:57,q2r:[5,57],q3:57,q4:57,q:[2,3,5,7,10,11,12,17,24,27,34,35,46,51,53,54,55,57,58,59,67,71,75],q_1:[7,34],q_:7,q_factordenom:17,q_factornum:17,q_factornum_l:17,q_i:[7,34],q_l:34,q_occurr:55,q_orient:55,q_r:34,q_reduce_fl:17,q_rewrit:55,q_scope:[5,71],q_u:34,q_with_bind:55,qarchimedean_power2_po:17,qarchimedeanexp2_po:17,qarith:[5,17],qarith_bas:17,qc:71,qc_scope:71,qcanon:11,qden:17,qden_cancel:17,qed:[3,5,6,8,9,12,13,14,17,24,29,32,34,36,38,40,42,51,52,54,57,58,59,60,62,64,66,67,72],qeq_from_part:17,qeval_formula:5,qextra:17,qhyp:55,qinv_neg:17,qinv_po:17,qinv_swap_neg:17,qinv_swap_po:17,qle_neq:17,qlt_leneq:17,qm:13,qmicromega:5,qmult_frac_l:17,qmult_inject_z_l:17,qmult_inject_z_r:17,qmult_le_lt_compat_po:17,qmult_lt_le_compat_nonneg:17,qnum:17,qnum_cancel:17,qopp_lt_compat:17,qpower_0_lt:17,qpower_1_l:17,qpower_1_le_po:17,qpower_1_lt:17,qpower_1_lt_po:17,qpower_decomp:17,qpower_decomp_po:17,qpower_le_1_increas:17,qpower_le_compat:17,qpower_le_compat_inv:17,qpower_le_compat_l:17,qpower_le_compat_l_inv:17,qpower_lt_1_increas:17,qpower_lt_compat:17,qpower_lt_compat_inv:17,qpower_lt_compat_l:17,qpower_lt_compat_l_inv:17,qpower_pos_lt:17,qr:46,qreduce_l:17,qreduce_num_l:17,qreduce_r:17,qreduce_zero:17,qround:17,qtautocheck:5,qtautochecker_sound:5,quad:5,quadrat:[2,17],qualid:[2,4,5,10,11,13,14,17,29,35,37,39,40,41,42,46,51,54,55,57,59,60,62,64,66,67,71,72,74],qualid_annot:[28,29,44],qualifi:[2,17,24,25,28,32,38,51,53,54,55,57,58,59,64,66,71],qualiti:[10,14,17],quantif:[2,3,4,13,14,17,24,26,27,28,60,67],quantifi:[8,14,17,24,25,26,28,34,39,44,57,58,62,67],quarkcool:17,quasi:57,quentin:17,queri:[13,17,25],query_command:[29,59,64],query_extra_dep:59,question:[25,34,54,55,57,60,66],quick:[13,17,24,27,54,57,66,74],quickli:[16,17,25,44],quicksort:24,quiet:75,quinn:17,quirk:52,quit:[2,3,11,13,17,25,34,42,54,55,57,60],quo_rem_un:57,quodlibet:[17,58],quot2:17,quot:[2,5,13,17,24,25,28,29,44,51,55,59,66,71,75],quot_rem:17,quot_rem_to_equ:[5,17],quotat:[17,24,25,66,75],quoted_str:53,quotient:[2,5,17,40,57,64],qux_plugin:53,qwit:5,qzero_eq:17,r0:[5,17],r1:[3,5,17,27,41,44,57,59],r2:[3,17,27,41,44,57,59],r3:57,r4:57,r:[2,3,5,7,9,11,13,14,17,24,27,28,34,35,37,41,44,51,53,54,57,58,59,60,64,67,71,72,75,77],r_1:3,r_2:3,r_dist:17,r_forest_size_complet:72,r_forest_size_correct:72,r_ifp:17,r_inj:17,r_item:57,r_pattern:57,r_plus_complet:[57,72],r_plus_correct:[57,72],r_prefix:57,r_s_inv:28,r_scope:[11,27,71],r_sqr:24,r_step:57,r_tree_size_complet:72,r_tree_size_correct:72,ra:13,rab:27,rabs_inv:17,race:17,raci:17,radboud:17,radd:11,radd_0_l:11,radd_assoc:11,radd_sym:11,radicalmax:7,radix3:71,radix3_ind:71,radix3_rec:71,radix3_rect:71,radix3_scop:71,radix3_sind:71,radix:[8,66],radixmorethanon:8,radixmorethanzero:8,radixnotzero:66,radziuk:17,railroad:24,railroadcross:24,rais:[2,3,10,13,17,29,35,54,55,64,72],raise_nat:10,rakam:[17,64],ralf:17,ralph:17,ram:17,ramachandra:17,ramkumar:17,ran:54,ranalysi:[17,24],ranalysis_reg:17,rand:17,randi:24,random:17,randomli:17,rang:[5,17,26,29,52,55,58,71],range_selector:54,rappli:[17,58],rard:77,rare:[11,17,66],rasmusson:17,rat:37,rat_bottom_nonzero:37,rat_irreduc:37,ratan:17,rather:[5,11,13,17,24,29,30,34,35,53,54,55,57,58,59,64,67,71],ratio:24,ration:[7,17,24,25,37,61,71],rational:[17,55,57],rauglaudr:[17,24],raw:[2,14,17,54,55,71],raxiom:17,rb:13,rbase:[11,17,24],rbox:12,rc:[17,24],rceil:5,rcl:34,rcomput:24,rdefinit:17,rdist:17,rdistr_l:11,rdiv:[3,5,27],rdiv_0_l:17,rdiv_0_r:17,rdiv_1_l:17,rdiv_1_r:17,rdiv_def:17,rdiv_diag:17,rdiv_diag_eq:17,rdiv_diag_uniq:17,rdiv_eq_compat_l:17,rdiv_eq_compat_r:17,rdiv_eq_reg_l:17,rdiv_eq_reg_r:17,rdiv_mult_distr:17,rdiv_mult_l_l:17,rdiv_mult_l_r:17,rdiv_mult_r_l:17,rdiv_mult_r_r:17,rdiv_neg_neg:17,rdiv_neg_po:17,rdiv_opp_l:17,rdiv_opp_r:17,rdiv_pos_cas:17,rdiv_pos_neg:17,rdiv_pos_po:17,re:[17,24,29,32,38,46,51,52,53,54,55,58,59,60,64,66],reach:[13,52,58],reachabl:71,reactiv:[8,17,59],read:[15,17,26,29,42,51,52,57,59,64,71,75],readabl:[2,17,24,29,53,57,64,71,75],reader:[3,11,24,29,31,42,57],readi:[17,51,57,60],readili:53,readm:[24,71],real:[2,3,7,11,24,25,34,46,53,55,66,67,71],realfield:11,realist:[2,42],realiz:[24,25,27,32],realli:[17,32,57],reappli:9,reason:[2,3,5,9,10,11,17,24,25,34,44,51,53,54,55,57,59,62,65,71,72,75,77],rebind:[5,17,52],rebuild:[13,17],rebuilt:53,rec:[2,17,24,35,54,55,75],recal:[46,55,64],recaptur:17,recdef:72,recent:[3,24,25,53,71],recheck:66,recip:[17,53],recogn:[2,4,5,8,11,17,24,29,34,46,51,52,55,62,67,71,75],recognit:[17,75],recommend:[4,8,13,14,15,17,32,35,46,51,52,53,54,55,57,58,59,60,64,66,67,72,74,75],recompil:[17,51,52,53,59,64],recomput:[34,53],reconstruct:[37,46],record:[2,3,8,10,11,12,13,14,17,24,25,30,33,34,42,54,55,57,59,60,62,67,71],record_definit:[4,13,30,34,37],record_field:[37,42],recov:[3,8,14,17,30,46,51,54,67],recover:55,recoveri:[8,17,52],rect:67,rectyp:17,recurr:25,recurs:[2,5,9,17,24,25,31,32,33,37,40,41,44,46,51,53,54,57,58,59,60,64,66,67,75,77],recursor:[2,17],red:[8,17,51,52,54,64,66],red_expr:[3,17,32,54,64],red_flag:17,redeclar:[13,17],redefin:[4,17,54,55,57,66,71,75],redefinit:[17,54,55],redesign:[17,24],redex:[2,17,25,31,34,64,71],redflag:17,redirect:[17,51,59,75],redo:[17,57,67],reduc:[3,7,8,10,11,12,13,17,24,26,31,32,34,36,37,40,41,44,51,53,57,58,59,60,64,66,67,71],reduce_and_try_to_solv:54,reduct:[2,3,9,10,11,12,17,25,26,30,32,36,41,44,46,51,53,57,58,67,77],redund:[17,24,43,46,57],redux:2,ref:[17,59],refactor:[17,64],refer:[2,3,4,5,8,10,13,14,16,24,25,28,29,31,32,34,35,36,37,38,39,41,42,44,46,50,51,52,53,55,57,58,60,62,64,66,67,71,72,74,75],referenc:[2,17,53,71],reference_occ:64,refglob:55,refin:[6,13,14,17,24,27,30,32,34,35,38,43,46,52,54,55,57,58,66,71],refl:[3,17],refl_eq:24,refl_equ:[3,17,57],reflect:[9,11,14,17,24,25,27,40,52,53,62,64,66,72,77],reflect_fals:57,reflect_tru:57,reflectf:40,reflectt:[40,57],reflex:[3,5,6,11,13,17,24,27,34,36,51,54,57,59,60,62,64,66,67,71],reflexion:24,reflexive_eq_dom_reflex:59,reflt:46,refman:17,refold:[17,64],reform:17,reformat:17,refrain:17,refresh:71,refrom:[17,51],refus:[2,3,64],refut:[25,57],regard:[3,14,17,51,58],regardless:[14,17,42,57,60,66],regener:53,regexp:[17,60],region:57,regist:[2,3,4,5,7,9,11,13,17,25,32,42,57,64,67,71,72],registr:[2,17,25],regress:17,regroup:17,regular:[9,10,13,17,36,46,51,55,57,60,64,75],regularli:17,rehaul:24,reifi:[5,17],reific:[7,17,64],reimplement:17,reimport:71,reinfer:44,reintroduc:[17,57],reject:[9,17,26,34,57,64,67,71],rel:[2,14,17,26,27,35,51,53,55,59,71],relat:[5,6,7,9,10,11,13,14,17,24,25,26,27,31,34,35,40,41,42,44,51,52,53,57,58,59,60,64,67,71,72,75],relation_definit:[3,13,17,59],relation_oper:17,relationclass:[3,17,64],relationship:[17,29],relaunch:17,relax:[2,17,30,44,53,57,60],releas:[13,15,17,24,25,52,53,57,63,74],releg:24,relev:[12,17,24,28,30,32,34,40,46,51,53,54,57,58,64,66,71],reli:[5,17,24,30,32,33,34,38,46,51,52,53,54,55,57,58,59,64,66,67,71],reliabl:17,relianc:17,reliev:24,reload:[51,52,59],reloc:24,relpr:17,rem:[5,17],remain:[2,3,9,11,13,14,17,24,34,36,39,41,42,44,46,52,57,58,64,66],remaind:[17,34,55],remap:71,remark:[4,17,24,25,32,34],remedi:[5,17],rememb:[17,52,57,58,75],remi:17,remind:[2,3,57],remot:17,remov:[2,3,4,5,11,14,17,24,29,31,37,41,46,51,52,53,55,57,58,59,60,66,67,71,72,74,75],remove_app:17,remove_con:17,remove_concat:17,remove_incl:17,remove_length_l:17,remove_length_lt:17,remove_remove_comm:17,remove_remove_eq:17,removelast_firstn_len:17,removelast_last:17,remzi:17,renam:[2,17,24,25,34,37,55,57,58,59,71,74],renard:[3,24],render:[17,24,75],renewcommand:75,renn:77,reopen:52,reorder:[17,25,52],reorgan:17,repair:[12,17],repars:[17,54],repeat:[3,17,25,43,44,52,55,57,58,59,66,67],repeat_app:17,repeat_con:17,repeat_eq_app:17,repeat_eq_con:17,repeat_eq_elt:17,repeat_to_concat:17,repeatedli:[17,31,57,71],repect:58,repetit:[25,54,60],replac:[2,3,4,7,9,10,11,17,24,25,28,31,32,34,37,41,43,44,46,51,52,53,54,55,57,58,59,62,64,66,67,71,74,75],replace_append_l:17,replace_append_r:17,replace_id:17,replace_replace_eq:17,replace_replace_neq:17,replace_with:55,replai:[11,57],replic:57,repo:53,report:[4,8,12,17,24,29,52,54,55,59,64,72,77],repositori:[17,53,63,74],repr:17,repres:[2,3,5,11,13,14,17,24,26,27,28,29,31,32,34,36,37,39,40,42,43,51,52,53,54,55,57,58,59,64,65,66,67,71],represent:[2,3,5,11,12,17,24,27,29,34,37,51,53,57,64,71],reprint:[17,66],reprocess:[52,54],reproduc:44,req:11,req_dec_t:17,req_em_t:17,request:[3,14,17,25,43,51,64],requir:[2,3,5,6,7,8,9,10,11,13,14,17,24,27,28,29,30,31,32,34,35,36,38,42,43,44,51,52,53,54,55,57,58,59,60,62,63,64,66,67,71,72,73,74,75],required_vo:51,rerun:5,resack0:60,research:[24,77],resembl:57,reserv:[17,25,27,29,35,40,54,57,59],reserv_list:44,reset:[2,17,24,29,30,34,40,41,46,51,52,54,59,72],resg0:60,resg1:60,residu:[17,57],resili:[17,25],resilient_command:17,resiz:17,resolut:[3,13,17,24,25,58,60,66,71,75],resolv:[9,13,14,17,35,43,52,55,57,58,59,60,64,66,67,71],resolve_tc:17,resort:[43,52,54,55,67],resourc:51,resp:[5,17,34,36,46,57],respect:[2,3,4,5,11,13,14,17,24,26,27,30,34,38,40,42,44,52,54,55,57,58,59,60,64,66,67,71,72,74,75],respons:[2,10,17,52,55,75],rest:[2,3,13,17,26,27,29,36,42,52,57,66],restart:[17,51,52,53,54,57,66],restart_tim:[17,54],restor:[17,29,54,57,66],restrict:[2,3,12,14,17,24,26,34,35,40,51,54,57,58,59,60,62,67,71],restructur:[17,24],result:[2,3,4,5,8,10,11,12,13,14,17,24,26,27,31,32,34,39,40,42,44,46,51,52,53,54,55,57,58,59,60,62,64,66,67,71,75],resum:17,ret:54,retain:17,retract:17,retri:54,retriev:[17,51,54,59,60,77],retro:17,retyp:17,reunion:77,reus:[14,17,41,57,58,59,63,64,66],reusabl:25,rev:[27,71],rev_con:17,rev_eq_app:17,rev_inj:17,rev_length:17,rev_nil:17,rev_repeat:17,rev_rev:17,rev_shiftin:17,revamp:17,revers:[7,15,17,25,27,34,41,57,58,60,66],reverse_coercion:[4,17],reversecoercionsourc:4,reversecoerciontarget:4,revert:[17,52,57,58,59],revgoal:17,review:[2,17,27],revis:[17,24,55],revisit:67,revolutionari:24,rew:[17,67,77],rew_iff_rev:57,rework:17,rewrit:[6,11,14,17,24,25,33,34,35,52,54,55,58,59,60,61,77],rewrite_occ:[3,64],rewrite_rul:10,rewrite_strat:[3,17],rewriterel:[3,17,57],rewritten:[3,9,11,24,30,46,57,58,64],rewrot:[11,17],rewstrategi:[3,17],rewstrategy0:3,rewstrategy1:[3,17],rexists_between:17,reynald:17,rfloor:5,rfrom:[17,51],rfunction:24,rgb:51,rge:[17,27],rge_gt_or_eq:17,rge_gt_or_eq_dec:17,rge_l:17,rge_lt_dec:17,rge_refl:17,rgeom:24,rgt:[17,27],rgt_le_dec:17,rgt_minus_po:17,rgt_or_l:17,rgt_or_not_gt:17,rh:[17,55,57,59],ri:[11,17,51],ribbon:52,rich:[9,17,57,73],richard:17,richer:[13,25],ricki:17,rid:[9,17,54,57],rideau:[17,57],rieg:17,rifrom:[17,51],right:[0,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,47,48,49,50,51,52,53,54,55,56,57,58,59,60,61,62,63,64,65,66,68,69,70,71,72,73,74,75,76,77],righta:71,rightarrow:[5,7,26,75],rightarrow_:[11,37],rigid:[3,10,13,14,17,24,60,72],rigor:[2,24],rin:17,rineq:17,ring31:17,ring:[7,17,24,25,27,37,61,62],ring_eq_ext:11,ring_mod:11,ring_morph:11,ring_plugin:[2,3,5,9,11,27,29,36,42,43,54,55,57,58,59,60,64,66,72],ring_polynom:11,ring_simplifi:[11,17],ring_theori:11,ringer:17,ringmicromega:5,rinv:[5,27],rinv_0_lt_contravar:17,rinv_div:17,rinv_eq_compat:17,rinv_eq_reg:17,rinv_inv:17,rinv_lt_0_contravar:17,rinv_mult:17,rinv_mult_simpl:17,rinv_neg:17,rinv_opp:17,rinv_po:17,rinv_r_simpl_l:17,rinv_r_simpl_m:17,rinv_r_simpl_r:17,ripault:17,rise:[13,24],risk:[10,17,24,51,59,66],rl:34,rle:[17,27],rle_epsilon:17,rle_gt_dec:17,rle_half_plu:17,rle_lt_or_eq:17,rle_or_gt:17,rle_or_not_l:17,rle_rinv:17,rlength:17,rlist:17,rlogic:17,rlt:[17,27],rlt_0_2:17,rlt_0_minu:17,rlt_ge_dec:17,rlt_half_plu:17,rlt_minus_0:17,rlt_monotony_contra:17,rlt_monotony_rev:17,rlt_or_g:17,rlt_or_not_lt:17,rlt_rminu:17,rmin_cas:17,rminu:[5,27],rminus_def:17,rminus_diag:17,rminus_eq_0:17,rminus_eq_compat_l:17,rminus_eq_compat_r:17,rminus_gt_0_lt:17,rminus_plus_distr:17,rminus_plus_l_l:17,rminus_plus_l_r:17,rminus_plus_r_l:17,rminus_plus_r_r:17,rmp:58,rmul:11,rmul_1_l:11,rmul_assoc:11,rmul_sym:11,rmult:[5,11,27],rmult_div_assoc:17,rmult_div_l:17,rmult_div_r:17,rmult_div_swap:17,rmult_gt_reg_r:17,rmult_inv_l:17,rmult_inv_m_id_r:17,rmult_inv_r:17,rmult_inv_r_id_l:17,rmult_inv_r_id_m:17,rmult_inv_r_uniq:17,rmult_neg_cas:17,rmult_neg_neg:17,rmult_neg_po:17,rmult_pos_cas:17,rmult_pos_neg:17,rmult_pos_po:17,rnm:58,ro:11,road:17,roadmap:17,robbert:17,robbiano:77,robert:[17,77],robin:[17,77],robinson:24,robust:[2,17,51,57,60,66,75],robustli:64,rocq:[3,4,6,8,9,10,11,12,13,14,15,17,24,26,28,29,30,31,32,33,34,35,36,37,38,41,42,43,44,45,46,50,52,54,55,58,59,62,63,64,65,66,67,73,76],rocqlib:59,rocquencourt:[17,24],rodi:17,rodolph:17,roi:[54,62,77],role:[17,26,33,42,55,71,75],romain:17,romega:[17,24],root:[3,17,25,27,46,51,59],ropp:[11,27],ropp_def:11,ropp_div:17,ropp_div_distr_l:17,ropp_eq_reg:17,ropp_minus_distr:17,ropp_neg:17,ropp_po:17,roquencourt:24,ros98:[9,77],rosetta:54,rosser:77,rotat:[24,54,57],round:[5,17,27,53],rousselin:17,routin:2,roux:17,row:[17,46],rplu:[5,27],rplus_0_l_uniq:17,rplus_eq_0:17,rplus_eq_r0:17,rplus_ge_reg_r:17,rplus_gt_reg_r:17,rplus_int_part_frac_part:17,rplus_le_lt_0_neq_0:17,rplus_minus_assoc:17,rplus_minus_l:17,rplus_minus_r:17,rplus_minus_swap:17,rplus_neg_lt:17,rplus_neg_neg:17,rplus_neg_npo:17,rplus_nneg_g:17,rplus_nneg_nneg:17,rplus_nneg_po:17,rplus_npos_l:17,rplus_npos_neg:17,rplus_npos_npo:17,rplus_pos_gt:17,rplus_pos_nneg:17,rplus_pos_po:17,rplus_sqr_eq_0_l:17,rpow:11,rpow_pow_n:11,rpower:17,rr:77,rrika:17,rs:17,rs_r:17,rsa:24,rsigma:24,rsqr:17,rsqr_def:17,rsqr_div:17,rsqr_inv:17,rstar:[17,24],rstep:57,rstrength:17,rsub:11,rsub_def:11,rta:77,rtac:55,rtauto:[17,62],rtran:58,rtrigo:24,rtrigo_calc:17,rudi:17,rudimentari:71,rug:55,rule:[3,4,5,11,12,13,14,17,24,25,29,32,33,35,36,37,39,41,42,44,46,51,53,54,55,58,59,60,62,66,67,77],run:[2,5,8,9,13,14,17,24,25,29,51,53,57,59,60,64,66,71,73],runbox:12,runner:17,runtim:[17,51,55,73],rushbi:77,russel:[9,17,24],rusu:72,rw_head_pattern:10,rw_pattern:10,rw_pattern_arg:10,rwf:27,ryan:17,s0:[43,46],s1:[3,30,38,57],s2:[3,30],s754_finit:27,s754_infin:27,s754_nan:27,s754_zero:27,s:[0,1,3,4,5,6,7,8,9,10,11,12,13,14,15,16,17,18,19,20,21,22,23,24,25,26,28,29,30,31,32,33,34,35,36,37,38,39,40,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,68,69,70,71,72,73,74,75,76,77],s_1:[7,34,35],s_2:[34,35],s_3:35,s_:[7,34],s_i:[5,7,34],s_item:57,s_j:34,s_k:34,s_nat:4,s_o_plus_inr_depr:17,sacerdoti:[3,17,24],safe:[2,11,17,34],safeimplicit:2,safer:[17,24],safeti:2,sai:[2,3,4,17,24,26,27,28,29,31,34,42,52,53,54,55,57,58,64,71,74],said:[3,4,17,26,34,36,42,44,55,59,71],saikawa:17,sakaguchi:17,sake:[35,55,66,71],salient:[17,24],sam:[17,77],same:[2,3,4,6,8,9,10,11,12,13,14,17,24,25,26,28,29,30,31,34,35,36,37,38,40,41,42,43,44,51,52,54,55,57,58,59,60,62,64,66,67,71,72,75],samel:71,samuel:[11,17,24],san:75,sandrin:77,santiago:17,satifi:34,satisfi:[3,4,5,11,13,14,17,30,34,35,54,55,59,64,67,71],satur:[5,17],save:[8,11,17,25,35,51,53,57,66],saw:24,sc:24,scale:[17,24,51,57,64,71],scan:54,scene:57,schedul:17,schema:24,schemat:[52,57],scheme:[2,11,17,24,25,26,27,34,37,40,46,51,57,59,62,77],scheme_kind:67,scheme_typ:17,scherer:17,schneider:17,schommer:17,schroeder:24,scienc:[24,77],scientif:[24,77],scinart:17,scope:[5,11,17,24,25,27,29,32,36,38,42,43,45,52,54,55,57,59,60,64,66],scope_kei:[40,55,59,64,71],scope_nam:71,scott:[17,24],scratch:52,screen:[17,52,59],screenshot:[52,66],script:[5,8,17,24,25,35,42,43,53,54,55,57,58,59,60,63,64,66,73],scrupul:17,scrutine:17,sdf:77,seamlessli:53,search:[2,3,4,5,7,13,17,24,25,42,44,51,52,53,61,62,64],search_item:59,search_queri:59,searchabout:[17,24],searchhead:17,searchiso:24,searchpattern:[17,24],searchrewrit:[17,24],seassau:17,sebastiaan:77,sec:[53,54,64],second:[2,3,4,8,9,10,11,13,15,17,24,25,26,28,35,37,38,40,42,44,51,52,53,55,57,59,60,64,66,67,71,75],secondari:[52,53],secondli:[2,17],section:[3,5,6,7,8,9,10,11,12,17,24,25,26,27,28,29,30,31,32,33,34,35,36,37,40,41,42,43,46,51,52,53,54,55,57,58,59,60,64,65,67,71,74],section_path:59,section_var_expr0:66,section_var_expr50:66,section_var_expr:[60,66],secur:51,sed:17,see:[2,3,4,5,7,8,9,11,12,13,14,17,24,26,27,28,29,30,31,32,33,34,35,36,37,38,39,40,41,42,43,44,46,51,52,53,54,55,57,58,59,60,62,64,66,67,71,72,74,75],seem:[2,5,17,71],seemingli:71,seen:[2,4,13,14,17,24,32,34,55,57,67,71],seg:24,segfault:[10,17],segment:[2,17,24,52,59,71],seldin:77,select:[8,13,17,25,35,37,41,42,52,53,54,55,58,59,60,64,66,67,71,75,77],selector:[8,17,25,43,53,58,59,64,66],self:[14,17,54,55,67,71],selfid:14,selfpid:14,semant:[3,11,13,14,17,24,25,26,29,35,36,39,41,44,53,54,57,58,71,77],semeria:17,semi:[4,11,17],semi_field_theori:11,semi_morph:11,semi_ring_theori:11,semicolon:[52,53,57],semidecis:24,semifield:11,semir:[11,17],sempti:12,sempty_ind:12,sempty_rec:12,sempty_rect:12,sempty_sind:12,send:17,sens:[4,24,26,30,54,55,57,71],sensibl:[14,24],sensit:[17,24,29,59],sent:52,sentenc:[17,24,29,36,52,54,55,57,59,75],sentence_1:24,sentence_n:24,sep:71,separ:[2,3,10,14,17,24,25,26,29,33,34,35,40,44,46,51,52,53,54,55,57,58,59,67,71,74],septemb:[17,24,77],seq:[12,13,30,46,55,57,67],seq_:17,seq_ind:[12,46],seq_length:17,seq_rec:[12,46],seq_rect:[12,46],seq_sind:[12,46],seqseri:24,sequenc:[2,3,5,17,24,25,27,28,29,30,46,51,57,58,59,60,64,66,71,75],sequent:[54,57,58,62,77],sequenti:[17,54,55,58,64],sergei:17,seri:[25,27,29,35,54,57],serial:[58,67],serif:75,seriou:[17,71],serv:[17,24,25,26,40,55,57,60],server:[17,52],session:[2,14,17,51,52,59],set1:26,set2:26,set:[0,1,3,4,5,6,7,8,9,10,11,12,14,15,16,17,18,19,20,21,22,23,24,25,27,28,30,31,32,33,34,35,36,38,39,40,42,43,44,45,46,47,48,49,50,51,52,53,54,55,56,59,61,62,63,64,65,67,68,69,70,71,72,73,74,75,76,77],set_diff_nodup:17,set_eq:3,set_map:17,set_p:34,seth:17,setistyp:17,setoid:[7,10,11,17,24,25,42,57],setoid_:[3,17],setoid_reflex:17,setoid_replac:[17,24,64,71],setoid_rewrit:[3,17,24,60,64],setoid_symmetri:17,setoid_theori:[11,17],setoid_transit:17,setoidchoic:17,setoidlist:17,setoidpermut:17,setoidtact:[17,71],setting_nam:[29,51],setup:[17,25],seventh:77,sever:[2,3,4,5,11,17,24,25,26,28,29,30,31,32,34,40,42,44,46,51,52,54,55,57,59,60,64,65,67,71,72,75,76],sf64mul:[27,36],sf:72,sf_1_neq_0:11,sf_sr:11,sfclassifi:17,sfdiv_def:11,sfinv_l:11,sfst:12,shachar:17,shachnev:17,shade:52,shadow:[14,17,44,66],shaji:17,shall:[2,17,24,26,31,34,39,42,57,71],shankar:77,shao:77,shape:[2,3,57],share:[2,11,13,14,17,24,28,29,34,46,51,52,53,57,59,60,64,67,71],she:[24,55],sheet:75,shelf:[17,66],shell:[51,53,57,59,75],shelv:[6,13,17,25,43,57,58,60],shelve_unifi:[17,58],shen:17,shengyi:17,shenlebantongi:17,shift:[17,52,57],shiftl:17,shiftl_lower_bound:17,shiftr:17,shiftr_upper_bound:17,shine:57,shinnar:17,ship:[17,66],shiwei:17,shortcut:[13,17,25,52,55,64,71],shorten:[17,28],shorter:[17,31,35,57,59],shortest:35,shorthand:[17,41,54,57,64],should:[2,3,9,10,11,12,13,14,17,24,26,28,29,30,32,34,35,40,41,42,44,46,51,52,53,54,55,57,58,59,60,62,64,66,67,71,74],shouldn:[53,54,75],show:[2,3,5,7,8,9,11,13,14,17,24,25,27,34,35,37,38,42,51,52,53,54,57,58,59,60,64,67,71],show_profil:17,show_zifi:5,shown:[5,9,13,14,17,27,29,31,34,37,38,42,43,51,52,53,54,57,58,59,60,66,71,75],shrink:[17,66],shuffl:57,sibut:17,siddharth:17,side:[3,10,13,14,17,24,25,27,32,34,35,38,43,52,54,55,57,58,60,62,64,67,71],sig2:[17,27,35,67],sig2_ind:27,sig2_rec:27,sig2_rect:27,sig2_sind:27,sig:[2,17,27,28,35,67,71],sig_ind:27,sig_rec:27,sig_rect:27,sig_sind:27,sigact:77,sigint:17,sigma:[14,17,37,67,71],sign:[5,8,11,17,29,36,46,52,53,60],signal:[2,8,17,57],signatur:[2,3,11,17,24,34,35,54,55,59],signature_scop:17,signaturet:17,signific:[17,24,51,63,66],significantli:[11,17,24,57,66],sigplan:77,sigt2:[17,27,67],sigt2_ind:27,sigt2_rec:27,sigt2_rect:27,sigt2_sind:27,sigt:[17,27,67,71],sigt_ind:27,sigt_of_prod:17,sigt_of_sigt2:17,sigt_prod_sigt:17,sigt_rec:27,sigt_rect:27,sigt_sind:27,sigtnot:17,sigurd:17,sile:17,silenc:[4,17,24,41,46,57,62,74],silent:[12,14,17,24,29,51,53,59,66,72],similar:[2,3,5,9,13,17,24,26,27,34,35,37,38,51,53,54,55,57,58,59,60,62,64,66,67,72,74,75],similarli:[9,10,13,14,17,26,28,36,38,42,44,46,52,53,54,55,57,62,64,71,75],simon:[17,77],simonbouli:17,simpl:[3,4,10,11,17,24,25,29,37,41,42,43,46,52,53,54,57,58,59,60,62,67,72],simpl_depind:67,simpl_rel:[3,17],simple_bind:67,simple_intropattern:[17,55,58,67,71,72],simple_intropattern_clos:58,simple_occurr:[58,60,64],simple_reserv:44,simple_tact:[24,54],simpler:[17,24,57,58,62,64],simplest:[55,57],simplex:17,simpli:[3,4,11,13,14,17,24,31,39,54,55,57,59,62,67,71,75],simplic:[35,54],simplif:[2,11,17,24,25,41,54,67],simplifi:[2,11,17,24,41,54,57,64,67],simplify_dep_elim:67,simplify_eq:[17,24,67],simplify_typ:54,simplify_type_eq:54,simplist:42,simpson:24,simul:[3,17,24,57,66],simultan:[3,17,24,25,26,30,32,34,42,53,57,58],sin3pi4:17,sin:17,sinc:[2,3,4,5,8,10,11,12,13,14,17,24,26,28,30,34,35,37,41,42,44,46,51,52,53,54,57,58,59,60,66,67,71,74,75],sine:17,singhal:17,singl:[2,3,4,13,14,17,24,25,28,29,30,34,35,37,40,44,46,52,53,55,57,58,59,60,64,66,67,71,75],single_z_r_r1_depr:17,singleton:[2,13,17,24,34,54,58],sint63:[17,36],sint63_scop:36,siromonei:[24,77],site:55,situat:[3,4,11,17,46,54,57,71],sixth:17,sizabl:57,size:[2,3,9,13,17,24,34,37,51,52,55,57,59,64,71,72],sizef:34,sizet:34,skeleton:9,skip:[8,17,41,42,46,51,53,54,57,58,64,66,67],skipn:17,skipn_length:17,skipn_non:17,skipn_seq:17,skipn_skipn:17,slant:75,slash:[17,57],slave:51,slexprod:17,slider:52,slight:[2,17,24,58],slightli:[3,17,24,35,51,52,54,55,57,58,67],slow:[3,11,17,53,54,55],slowdown:17,slower:[17,51,60,62],slowest:53,slowli:54,slrnsc:17,small:[3,5,8,11,14,17,25,26,27,33,34,39,42,44,52,53,57,64],smaller:[3,11,14,17,32,33,34,53,58,62,67,72],smallest:[3,5,27,34,67],smart:17,smart_glob:71,smarter:17,smit:17,sml:24,smooth:[17,24,57],smorph0:11,smorph1:11,smorph_add:11,smorph_eq:11,smorph_mul:11,snd:[17,24,27,35,42,46,71],snd_list_prod:17,snippet:[55,75],snoc:67,snyke7:17,so08:[13,77],so:[2,3,4,7,8,9,10,11,12,13,14,17,24,26,27,29,31,32,34,35,36,37,38,44,46,51,52,53,54,55,57,58,59,60,62,64,66,67,71,73,74,75],societi:77,socket:17,soegtrop:17,soft:[25,72],softwar:[17,24,25,59,77],sogetrop:17,solut:[3,5,13,17,42,44,58,59,63,67],solv:[2,3,5,7,11,13,17,24,25,39,42,44,57,60,61,62,64,67],solvabl:[17,58,62],solve_constraint:66,solve_iso:54,solve_iso_ex1:54,solve_iso_ex2:54,solve_perm:54,solve_type_eq:54,solver:[9,17,25,65],some:[3,4,5,6,8,9,10,11,12,13,14,17,24,25,26,28,29,30,31,32,34,37,38,40,41,42,44,45,46,51,52,53,54,55,57,58,59,60,61,62,63,64,66,67,71,72,73,75],some_class:17,some_const:42,some_expr:17,some_term:17,somehow:46,someon:17,someth:[17,31,52,53,54,55,59,64],sometim:[14,17,24,25,31,34,46,53,54,55,57,59,60,66,67,71],somewhat:[55,64,71],soon:[8,9,17,24,42,52,54,57],sop:24,sophia:[17,24],sort:[0,1,2,3,4,5,6,7,8,9,10,11,12,13,15,16,17,18,19,20,21,22,23,24,25,26,27,28,29,30,31,32,33,35,36,37,38,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],sort_famili:[67,72],sortclass:[4,17,57,71],sorted_sort:17,sotaro:17,soubiran:17,sought:46,soukouki:17,sound:[2,17,34],sourc:[2,4,5,14,24,25,51,52,53,55,57,59,71,73],source_date_epoch:17,soz07:[9,77],sozeau:[3,9,14,17,77],sp1:17,space:[3,17,29,52,53,57,59,66,71,74,75],space_overhead:51,span:17,spanjel:17,spawn:[17,54],speak:[5,11],spec:[5,17],spec_float:27,special:[2,3,4,9,12,13,16,17,24,25,27,28,29,34,51,52,53,54,55,59,60,64,66,67,71,75],specialist:17,specif:[2,3,5,9,11,24,28,31,32,34,35,36,39,40,42,51,52,53,55,57,58,59,60,61,64,66,67,71,77],specifi:[2,3,4,5,6,9,11,13,17,24,25,27,28,29,32,34,35,36,37,40,41,43,44,46,51,52,53,54,55,57,58,59,60,62,64,66,67,71,72,75],spectacular:24,speed:[3,13,17,24,34,64],spell:17,spent:[17,51,53,54],sphinx:17,sphinx_rtd_them:17,sphinxcontrib:17,spin:17,spirit:[17,34,55],spite:17,spitter:17,spiwack:17,splay_ar:17,split:[2,17,25,27,29,34,42,51,54,57,58,60,66,67,75],split_combin:17,split_length_l:17,split_length_r:17,split_rab:27,split_rmult:27,splitabsolu:24,splitat:17,splitrmult:24,spontan:57,spot:55,spr1:12,spr2:12,spread:53,spring:24,springer:77,sprod:12,sprop:[0,1,2,3,4,5,6,7,8,9,10,11,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],spuriou:[4,17,57,71],spurious:17,sqrt:[17,27,59],sqrt_inv:17,sqrt_iter:59,squad:2,squar:[5,17,24,44,54,59,71,75],squash:[12,14,17],squash_ind:14,squash_prop_rect:14,squash_prop_srect:14,squash_sind:14,sr:10,sradd_0_l:11,sradd_assoc:11,sradd_sym:11,src:[4,53],srdistr_l:11,srefl:[12,46],sring_eq_ext:11,srinivasan:17,srmul_0_l:11,srmul_1_l:11,srmul_assoc:11,srmul_sym:11,ssig:12,ssnd:12,ssort:4,ssr:[17,57,59,66],ssr_binder:57,ssrautoprop:57,ssrbool:[17,57],ssreflect:[0,1,2,3,4,5,6,7,8,9,10,11,12,13,14,15,16,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,58,59,60,61,62,63,64,65,66,67,68,69,70,71,72,73,74,75,76,77],ssreflect_plugin:57,ssrewrit:17,ssrfun:[17,57],ssrhave:[17,57],ssrident:57,ssripat:57,ssripat_scop:57,ssrmatch:[17,57],ssrmatching_plugin:57,ssrnat:57,ssroldrewritegoalsord:57,ssrrewrit:57,ssrsearch:17,ssrsyntax:57,sstuff:4,stabil:17,stabl:[8,17,24,53],stack:[17,25,41,54,55,57,59,71],stage:[17,34,42,55,66],stai:[2,27],stale:17,stalmarck:[2,24],stand:[5,10,17,24,26,28,34,53,71],standalon:[17,51],standard:[2,3,5,9,14,25,29,35,36,40,51,52,53,54,58,59,62,64,65,66,67,72,73,74,75],stanza:53,star:[17,60,62],starred_ident_ref:66,start:[2,3,8,9,13,17,24,25,26,27,29,32,34,35,37,40,41,42,44,46,52,53,54,55,58,59,60,64,66,67,71,74,75],start_coq:53,start_profil:17,startclass:17,startup:[12,51,53,60],stat:66,state:[2,3,5,7,8,11,13,17,24,25,27,29,31,32,37,51,52,54,55,57,58,59,62,64,67,71],statement:[8,9,17,24,28,32,33,41,42,44,51,57,58,59,64,66,67,71],station:17,statist:[5,17,66],statu:[8,12,13,14,17,51,52,53,54,57,71],std:[17,55],stdlib:[2,3,5,6,9,12,14,17,27,28,35,36,51,53,54,55,57,58,59,64,66,67,71,75],stdout:[17,75],steckler:17,stefan:17,stell:17,stem:17,stengl:17,step:[3,5,7,11,13,17,24,25,26,29,41,51,52,53,54,58,60,64,65,67],stepanenko:17,stephan:17,stepl:[17,64],stepr:[17,64],stick:55,sticki:24,still:[2,3,7,9,10,13,17,24,29,32,34,36,37,38,42,44,46,51,53,54,57,58,59,60,64,66,67,74],stm:17,stmaryrd:75,stock:17,stolz:17,stone:54,stop:[3,5,12,17,24,32,38,52,54,57,71],stop_profil:17,store:[17,27,52,53,57,59,60],stori:30,storm:17,str:[0,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],straightforward:[3,55],straightforwardli:3,strat:3,strategi:[7,9,13,17,24,25,26,55,57,59,60,71,77],stratego:[3,77],strategy_level:[64,71],strategy_level_or_var:[64,71],stratif:24,stream:[0,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],stream_eta:30,stream_ext:30,streamlin:[17,24],strength:24,strengthen:[17,35,57,67],strict:[2,5,13,14,17,24,25,31,39,41,42,54,57,58,59,60,66,71],stricter:[13,14,17],strictli:[8,11,14,17,41,57,71],strictprop:[12,17],strikeout:66,string:[2,11,13,14,17,25,29,40,42,51,53,54,55,57,59,64,66,74,75],string_as_ot:17,string_get:36,string_length:36,string_scop:[17,42,71],string_typ:36,stringsyntax:17,strip:[17,58],strong:[17,24,27,31,34,64,67,77],strong_induction_l:17,stronger:[3,12,17,34],strongli:[11,15,17,34,35,44,53,54,57,59],strub:17,struct:[0,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],structur:[2,3,4,8,9,13,17,24,25,27,32,34,35,36,37,38,40,44,45,53,54,58,59,66,67,71,72,77],stt:12,stuck:[12,13,17],studi:[24,31],stuff2:53,stuff:[24,53,75],style:[6,17,24,25,30,37,52,55,57,62,67],suarez:24,sub:[2,4,8,17,27,36,41,46,51,53,54,57,59,60,67,71],sub_equ:72,subcas:[40,75],subclass:[4,10,13,27,39,42,59],subcompon:[17,51],subdir:[17,51,53],subdirectori:[17,27,51,53,59,60],subequ:67,subexpress:[54,58,71],subgoal:[5,11,13,17,24,25,27,54,57,58,60,62,64,67],subgraph:[14,17],subject:[10,17,25,26,30,31,50,51,72],sublemma:17,submak:53,submit:[24,27],submodul:[17,35],subnk:57,subnn:57,subpackag:59,subpart:54,subpattern:[25,54,55],subprocess:17,subproof:[17,34,66,67],subrel:[17,25],subscript:29,subsecond:53,subsect:[17,24,34,42,75],subsequ:[8,14,17,29,37,38,51,54,55,58,59,66,67,71],subsequent_lett:29,subset:[5,9,17,24,25,34,39,44,55,57,58,66,71,77],subset_bi:71,subst:[0,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],substitut:[10,11,17,24,25,26,34,38,46,51,55,57,58,64,67,71],substr:[17,59],substructur:[17,25],subsum:[17,57],subsystem:[17,24],subterm:[3,9,10,11,17,24,25,31,34,41,54,55,57,58,59,64,66,67,71,72],subtim:51,subtitl:75,subtract:[5,57],subtyp:[4,9,14,17,25,31,35,39,77],succ:[2,24,54,59,64],succ_doubl:17,succ_po:17,succe:[2,3,13,17,25,44,46,51,55,57,58,59,60,62,64,66],succeed:[3,17,54,59,72],success:[2,3,4,5,13,17,24,25,34,51,52,55,57,59,60,62,64,66,67,74],successfulli:[13,51,52,54,57,62,63],successor:[24,34,39],succinct:55,suchthat:[6,17],suddenli:55,sudha:17,suff:[17,25],suffic:[52,57],suffici:[3,5,11,13,53],suffix:[3,17,35,51,52,53,54,57,59,71,75],sugar:[2,7,17,28,54,55,59,77],suggest:[11,17,24,25,34,51,52,53,57,66],suit:[2,17,53,57,58,63],suitabl:[17,41,52],sum:[11,17,24,27,35,38,40,55,62,67,71],sum_:[5,7,57],sum_ind:[24,27,71],sum_inequa_rle_lt_depr:17,sum_rec:[27,71],sum_rect:[27,71],sum_sind:[27,71],sumbool:[2,27,46,71],sumbool_ind:27,sumbool_rec:27,sumbool_rect:27,sumbool_sind:27,sumlist:57,summar:[11,51,57,66],summari:[25,46,51,75],summaris:57,summat:57,summer:24,sumor:[27,71],sumor_ind:27,sumor_rec:27,sumor_rect:27,sumor_sind:27,sumxxx:57,sun:24,sunit:12,sunit_rect:12,sup:24,superclass:25,superfici:10,superflu:[17,24],superieur:17,superpos:46,superposit:46,supersed:17,supervis:[17,24],supplement:17,suppli:[17,37,57,62],support:[2,3,4,5,6,8,9,11,13,14,17,24,25,27,30,32,34,35,36,37,40,41,42,44,51,53,54,55,57,59,60,62,63,64,66,71,72,74,75,76],suppos:[3,9,17,51,55,57,64],suppress:[57,75],sure:[2,4,17,35,52,53,58,71],suresn:24,surgic:57,surject:[11,37],surma:17,surpass:17,surpris:58,surround:[3,17,44,57,59,71],survei:[24,25],surviv:[17,24,60,71],suspend:[13,17,66],sustem:59,sven:17,swap:[2,17,54,57,58],swasei:17,sweet:55,sy:53,syllabu:24,sylvain:[17,77],sylvi:24,sym:[3,17,44],sym_equ:[17,57],symbol:[2,3,11,14,17,24,25,27,28,29,31,41,42,43,46,57,59,60,62,64,67,71,75,77],symlink:17,symmetr:[3,17,24,31,59,64,71],symmetri:[3,17,24,34,44,57,60,64],symposium:[24,77],symptom:17,syn_valu:54,sync:17,synchron:[17,24,52],synonym:[17,29,37,51,57,58,64],synopsi:[25,53],syntact:[2,3,11,17,24,25,26,27,28,29,30,31,34,35,37,39,41,57,58,59,64,66,71,74],syntax:[2,4,5,6,8,9,11,13,14,25,26,27,30,32,34,35,37,39,40,41,42,43,45,51,52,53,58,59,60,63,64,66,75,77],syntax_modifi:[17,71],synth:[46,59],synthes:[4,17,24,27,28,42,46,77],synthesi:[17,24,44],synthesis:2,synthesiz:46,synthet:24,system:[3,8,9,11,17,24,25,26,27,28,29,32,33,34,38,39,46,51,52,53,54,55,57,59,60,62,71,73,77],systemat:[17,24,44,55,57,64],t0:57,t1:[3,13,17,34,42,46,57],t2:[17,34,42],t:[0,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,65,66,67,68,69,70,71,72,73,74,75,76,77],t_0:26,t_1:[3,26,31,34,35],t_2:[26,31,34,35],t_:[26,34],t_h:66,t_i:34,t_ind:[17,35],t_k:26,t_m:34,t_n:[3,26,34,66],t_q:34,t_rec:35,t_rect:35,t_scope:[17,71],t_sind:35,t_tauto_intuit:54,tab:[17,29,52,53],tabareau:[3,17,77],tabl:[2,3,4,16,17,24,25,27,35,37,38,46,51,53,54,55,57,59,67,71,75],tableau:24,tableofcont:75,tablog:24,tabul:[17,24,57],tac1:17,tac2:17,tac2alg_constructor:55,tac2def_bodi:55,tac2pat0:55,tac2pat1:55,tac2rec_field:55,tac2rec_fieldexpr:55,tac2rec_fieldpat:55,tac2typ_def:55,tac2typ_knd:55,tac2typ_prm:55,tac:[0,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],tacdef_bodi:54,tacexpr:43,tacl:54,tacmach:17,tacn:71,tactic1:57,tactic:[7,8,9,10,13,16,25,26,29,30,31,32,33,34,35,38,40,41,46,51,52,53,59,62,65,66,73,75],tactic_arg:54,tactic_atom:54,tactic_failur:55,tactic_invoc:58,tactic_list_sep:54,tactic_then_loc:71,tactic_valu:54,tacticm:57,tacticn:57,tacvalu:52,tag:[17,24,51,52,57,66],tail:[17,24,27,46,54,55,57,60,71],tail_add:59,tail_addmul:59,tail_mul:59,tailor:11,taint:51,taiwan:77,takafumi:17,takahashi:77,take:[2,3,5,8,11,12,13,17,24,26,27,28,29,31,32,37,40,41,42,46,51,52,53,54,55,57,58,60,62,64,66,67,71,75],taken:[2,9,13,17,24,34,36,42,44,53,57,64,67,71],talia:17,tame:77,tan:77,tan_atan:17,tan_inj:17,tan_is_inj:17,tanaka:17,tankink:17,tapsoft:24,target:[4,11,17,25,51,58,71],tarski:24,task:[17,57,75],tassi:[8,17,42,57,77],tau:67,tauto:[5,17,24,34,54,62],tauto_gen:54,tauto_intuitionist:54,tautolog:[11,17,24,54,62],taylor:77,tctl:24,teach:17,team:[17,24],tebbi:17,tech_rgt_minu:17,tech_rplu:17,tech_single_z_r_r1_depr:17,technic:[8,17,27,34,44,51,57,71,77],techniqu:[5,9,30,42,57,59,62,67],tediou:[24,34,53,57,67],tej:[17,58],tel:77,telecom:24,telescop:17,tell:[2,3,11,17,24,34,41,42,44,46,51,55,57,60,64,67,71,75],templat:[13,17,25,30,37,40,66],tempor:24,temporari:[2,14,17,24,57],temporarili:[17,53,57,59,66,71],ten:24,tend:[14,57],teo:77,term0:[29,37,55,58,71],term100:[29,40,46],term10:[17,29,32],term1:[28,29,37,44,57],term2:57,term:[2,3,4,9,10,11,12,13,14,17,24,25,27,28,29,30,31,32,33,34,35,36,37,38,39,40,41,42,43,44,46,50,53,57,58,59,60,62,63,66,67,72,75],term_appl:[28,29,37,44,64],term_cast:[29,32],term_cofix:[17,29,30,54],term_evar:[29,43],term_explicit:[29,44],term_fix:[17,29,34,54],term_forall_or_fun:[17,28,29],term_gener:[29,44],term_i:57,term_if:[17,29,46],term_ind:67,term_let:[17,29,32,38],term_ltac:[29,54],term_match:[29,40],term_project:[29,37],term_rec:67,term_record:[29,37],term_rect:67,term_scop:[29,71],term_sind:67,termin:[2,9,17,24,25,27,29,30,32,34,35,38,51,52,55,59,60,66,71,72],terminolog:[24,55],termn:57,termvh:57,ternari:17,terrass:77,territori:52,test:[2,3,4,9,10,11,13,17,24,25,29,30,34,42,46,55,57,58,59,66],test_algebra:42,test_algebraic2:42,test_big_nest:57,test_ind:57,test_sind:57,testbit:[17,59],testbit_div2:17,testbit_eqb:59,testbit_even_succ:17,testbit_fals:59,testbit_nat:59,testbit_odd_succ:17,testbit_spec:59,testbit_tru:59,testcompil:[2,17],tetlei:17,tew:17,tex:[17,53,75],texa:24,texmac:75,text:[17,24,27,51,52,53,57,59,66,71,75],text_:75,textbook:57,textgreek:75,textsf:[0,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],textsl:75,texttt:3,textual:[17,46,71],tgt:53,th:[17,27,30,34,40,57,58,66,67,77],than:[2,3,5,8,11,12,13,14,17,24,29,30,31,34,35,37,43,44,46,51,52,53,54,55,57,58,59,60,62,64,66,67,71,72,73,75],thank:[2,5,12,17,24,34,42,55,57,64,71],the_cmp:42,thei:[2,3,4,6,7,8,9,10,11,12,13,14,15,17,24,25,26,27,28,29,30,31,32,34,35,36,37,38,39,41,42,43,44,45,46,51,52,53,54,55,57,58,59,60,64,66,67,71,72,73,74,75],them:[2,3,9,10,11,13,14,17,24,26,27,28,31,34,35,37,38,40,41,42,43,44,46,51,52,53,54,55,57,58,59,60,62,64,66,67,71,72,73,75],theme:[24,52],themselv:[3,13,14,17,26,35,37,39,41,42,53,57,59,64,71],theorem:[2,5,7,8,11,12,17,24,25,27,29,32,33,35,37,38,42,43,51,52,57,59,60,62,65,66,71,73,74,75,77],theorem_nam:66,theoret:[2,17,24,31,39,77],theori:[3,4,5,11,17,24,25,26,27,28,29,39,42,46,51,53,57,58,60,62,67,71,77],theorylist:17,thereaft:[34,59],therebi:59,therefor:[2,17,29,31,37,52,53,57,58,62,72,73],therein:53,thereof:17,theri:[17,24],thesi:[24,77],thi:[2,3,4,5,6,7,8,9,10,12,13,14,15,17,24,25,26,27,28,29,30,31,32,33,34,35,36,37,38,39,40,41,42,43,44,45,46,50,51,52,53,54,55,57,58,59,60,61,62,63,64,65,66,67,71,72,73,74,75,76],thierri:[17,24,34,77],thing:[17,52,54,55,59,67,72],think:[55,66],third:[2,3,17,25,40,41,44,51,52,53,54,57,58,59,75],thirdli:17,this_scop:57,thisextrafil:53,thm:24,thm_token:[32,59],tho:17,thoma:17,thoroughli:[17,55],those:[2,3,5,10,11,12,17,24,26,33,34,35,37,43,46,52,53,54,55,57,58,59,60,62,64,66,67,71,72],though:[2,8,9,17,24,29,34,35,37,46,51,53,54,55,64,67,71],thought:[9,26,29,63],thread:17,three:[2,4,9,11,17,24,25,34,40,52,53,54,57,59,60,67,71],threeintropatternscombin:58,threshold:[8,17,64,71],throttl:77,through:[3,4,12,17,24,27,28,29,30,32,34,35,36,37,46,52,53,54,55,57,58,59,60,64,65,66,67,71,72,73,74],throughout:[17,29],thrown:2,thu:[2,3,4,5,10,12,17,24,32,34,42,43,46,51,53,54,55,57,58,59,60,64,66,67,71,72,75],thumb:[51,67],thunk:[17,55],ti:[13,57],tie:64,tight:71,timani:17,time1:53,time2:53,time3:53,time:[2,3,5,8,9,11,12,13,14,17,24,25,27,28,29,32,34,36,37,41,42,44,46,52,55,57,58,59,64,66,67,71],time_constr1:54,time_constr:[17,25],time_of_pretty_build_fil:53,timeout:[12,17,25,59,64],timer:54,times_sym:17,timing_fuzz:[17,53],timing_include_mem:[17,53],timing_r:[17,53],timing_sort_bi:[17,53],timing_sort_by_mem:[17,53],timothi:17,timur:17,tip:[17,60],titl:[17,52,75],tj:57,tl:[0,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],tl_map:17,tm:13,tmp:17,tn:[3,13,17,57],to_bit:59,to_bits_of_bit:59,to_constr:55,to_eq:42,to_euclidean_division_equ:[5,17],to_euclidean_division_equations_with:17,to_intro_pattern:17,to_l:42,to_list:17,to_list_append:17,to_list_con:17,to_list_const:17,to_list_exist:17,to_list_fold_left:17,to_list_fold_right:17,to_list_foral:17,to_list_forall2:17,to_list_hd:17,to_list_in:17,to_list_inj:17,to_list_last:17,to_list_map:17,to_list_nil:17,to_list_nil_iff:17,to_list_nth_ord:17,to_list_rev:17,to_list_rev_append:17,to_list_rev_append_tail:17,to_list_tl:17,to_n:17,to_nat:17,to_num_uint:71,to_po:17,to_preterm:17,to_str:[17,55],to_uint:71,to_uint_dec:71,tobia:17,toc:[17,75],todd:75,todo:17,togeth:[2,3,9,17,24,25,27,31,34,35,43,53,54,55,57,66,71,75],toggl:[46,52],toggleabl:17,toi:57,token:[17,29,42,51,52,53,54,55,58,59,66,71,75],toler:17,tolmach:77,tom:17,toni:17,too:[8,9,11,17,54,55,57,58,67,71],took:[17,24],tool:[11,14,25,29,51,52,53,54,57,59,66,71,72,75,77],toolbar:52,toolbox:[3,17],toolchain:[17,51],tooltip:[17,52],top:[3,8,10,12,13,14,17,24,25,27,29,35,37,46,51,52,53,54,55,57,58,59,64,67,71,73,75],top_heap_word:66,topbin:17,topdown:3,topfil:17,toplevel:[2,10,14,17,24,25,27,29,35,44,46,51,52,53,55,57,58,59,60,64,71,72,74],toplevel_selector:[17,29,54,58],toploop:17,toset:[14,17,34],total:[51,53,54],toto:51,toulous:17,toward:[4,17,27,53],tphol:77,trace:[11,13,17,25,32,51,53,57,58,59],track:[17,24,51,53,55,57],tracker:[17,54],tract:77,tractabl:12,tradit:[17,24,51,63],trager:17,traian:17,trail:[17,25,57,74,75],trailer:75,tran:[3,17],trans_equ:57,transact:[64,77],transfer:24,transform:[3,4,11,17,29,57,58,66,67,77],transit:[3,7,8,13,14,17,24,25,26,35,41,44,51,54,57,58,59,60,64,66,74],translat:[2,3,17,24,25,33,41,45,57,71,75],transpar:[3,4,6,9,14,17,24,25,31,32,35,37,41,51,54,55,57,59,60,64,66,67,75],transparentst:17,transport:[12,17],transposit:17,trap:24,travers:[3,17,57,58,67],traverso:77,travi:17,treat:[9,12,13,17,29,46,53,54,57,59,60,62,64,67,71,72],treatment:[2,9,17,40],trece:57,tree:[0,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,68,69,70,71,72,73,74,75,76,77],tree_forest_ind:67,tree_forest_mutind:67,tree_forest_mutrect:67,tree_forest_rec:67,tree_forest_rect:67,tree_ind:[34,67,72],tree_rec:[34,67,72],tree_rect:[34,67,72],tree_sind:[34,67,72],tree_siz:[34,72],tree_size_equ:72,tree_size_ind2:72,tree_size_ind:72,tree_size_rec:72,tree_size_rect:72,treinen:17,tri:[3,4,5,9,13,14,17,34,35,41,46,52,53,54,55,57,58,59,60,62,66,67],triangl:[10,52],triangleright:[26,31],triangleright_:[0,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],trick:[24,55,57,58,72],trickeri:55,tricki:[24,57],trickier:54,trigger:[13,17,25,29,44,54,55,57,60,71],trigonometr:[17,24],trii:[0,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],trili:17,trim:74,trivial:[12,13,14,17,34,46,53,54,55,57,58,60,66,67],trm:54,troubl:[17,54,64,67],true_sub:17,truli:[17,57],trunc:17,truncat:[17,57],trunk:17,trunov:17,trust:[24,33,36,73],truth:[17,54,57],tryif:[17,25],ts:46,tt:[5,13,14,17,27,40,46,54,57],tt_h:66,tt_n:66,tune:[17,38,42,64],tupl:[9,17,37,42,46,55,57,58],turn:[2,8,10,12,13,14,17,24,27,29,32,37,41,42,44,46,51,52,54,55,57,58,59,64,66,67,71],turner:17,tutori:[17,25,63,74,77],tv:2,tweak:17,twice:[17,34,51,59,64,66],two:[2,3,4,5,8,9,10,11,13,14,15,17,24,25,26,27,29,30,31,34,36,37,38,40,41,42,44,46,51,52,53,55,57,58,59,60,63,64,66,67,71,74,75],twofold:28,twoi:57,tx:57,txt:[17,24,53],ty:[54,57],typ:[17,24,34],typabl:[2,4,34],type1:35,type2:35,type:[0,1,5,6,7,8,9,11,12,13,14,15,16,18,19,20,21,22,23,24,25,27,29,31,33,36,39,41,42,43,45,47,48,49,50,51,52,53,56,58,60,61,62,63,64,65,66,68,69,70,72,73,74,75,76,77],type_ind:67,type_of:17,type_rec:67,type_rect:67,type_scop:[13,14,17,25,34,44,46,52,54,58,66,67],type_sind:67,type_term:[17,25],typeabl:3,typecheck:[9,17,41,51,55,58,59,64,66],typeclass:[3,4,5,7,17,25,35,37,38,44,45,58,60,64,66,71],typeclass_constraint:44,typeclass_inst:[13,17,60],typed:[10,55],typeexpand:2,typeset:[17,75],typic:[2,4,6,12,14,17,24,28,29,30,34,35,44,46,51,53,55,57,58,59,60,64,67,71],typo:[17,44],u05d0:17,u0:[10,14,46],u1:[10,13,14,17,57],u2:10,u:[3,4,9,10,14,17,24,26,27,31,34,35,38,39,41,46,53,54,55,57,58,62,64,67,71],u_0:26,u_1:[26,31,34,39],u_2:31,u_:34,u_i:[26,34],u_m:26,u_n:39,ubiquit:57,uconstr:[17,54,71],ui:[17,51],uint63:[17,27,36],uint63_scop:[36,71],uint:[17,59,71],uint_scop:17,uintdecim:71,uinthexadecim:71,uip:[14,17,25,46,59],uip_nil_l:17,uip_nil_nil:17,uip_nil_r:17,uip_none_l:17,uip_none_non:17,uip_none_r:17,uip_refl_nat:67,uj:57,ultim:11,um:[13,57],un:77,unabl:[3,14,34,43,46,53,57,58,59,66,67],unabletounifi:17,unambigu:[17,27,32,44,53,59],unappli:17,unari:[2,3,26,29,34,64],unavail:17,unavoid:57,unbound:[13,14,17,54,55,58],unbox:54,uncapit:17,uncaught:[17,55],unchang:[17,54,57,58,60,64,66],uncheck:59,unclear:[3,10,54],uncom:52,uncommon:17,uncon:17,uncondition:17,uncurri:17,undecid:[29,30],undeclar:[14,17],undefin:[17,28],undelimit:[17,59,71],undeprec:17,under:[5,9,11,17,25,32,40,44,46,52,53,54,55,59,64,66,67],under_rel:17,underli:[9,11,17,24,26,54,57,67,71],underlin:[51,52,66],undermin:57,underscor:[14,17,29,37,44,51,71,75],understand:[3,5,10,12,15,17,24,25,29,33,51,53,54,55,59,60],understood:[17,32,34,36,60,71,75],undertaken:24,undesir:64,undetect:[17,46],undetermin:[57,66],undif:66,undiscrimin:[17,60],undo:[11,17,52,54,58,59,66],undocu:[17,24,59],undon:52,unduli:17,uneed:58,unend:71,unequ:17,uneven:17,unexpect:[17,24,44,53,55,71,73],unexpectedli:54,unfocu:[17,66],unfocus:[17,34,55,59,66,67],unfold:[5,9,13,14,17,24,25,27,31,32,34,37,54,55,57,60,62,66,71],unfold_nth_error:17,unfortun:[3,5,17,42,46,57],unguard:30,unibo:24,unicod:[17,25,75],unicode_id_part:29,unicode_lett:29,unicoq:53,unif:[3,10,13,17,24,25,37,40,42,43,54,60,64,71],unifi:[3,12,13,14,17,34,41,42,43,54,57,58,64,66],uniform:[4,17,24,34,40,44,54,55],uniformli:[17,24,51],uninform:17,uninstal:[17,25],uninstanti:[43,44,54,58,67],unintend:57,unintendedli:17,uninterest:57,uninterpret:[17,62],uninterrupt:17,union:[3,13,17,54,59,66,77],union_compat:3,union_mor:3,uniqu:[2,3,12,13,17,24,27,31,35,38,57,59,67,71],unit:[2,12,13,14,17,27,34,40,46,53,54,55,57,62,64,71],unit_eqdec:13,unit_ind:27,unit_monoid:14,unit_rec:27,unit_rect:27,unit_sind:27,uniti:11,univ:17,univ_annot:[10,14,29,37],univ_constraint:14,univ_decl:[10,14,28,35],univ_level_or_qu:14,univ_name_list:59,unival:17,univers:[3,4,8,9,12,13,17,24,25,26,27,28,29,30,31,32,33,34,37,39,40,44,46,51,54,57,59,62,66,67,71,77],universe_expr:39,universe_nam:[14,39],unix:[17,24],unjustifi:17,unkei:57,unknown:[17,29,42,43,58,60,66,71],unless:[2,3,13,14,17,29,40,41,42,44,51,52,57,58,64,71,72,75],unlik:[10,13,17,24,30,39,52,54,55,57,58,59,60,64,67,71],unload:17,unlock:25,unmaintain:17,unmatch:58,unmodifi:52,unnam:[17,44,52,57,66,71],unnamed_coqscript_:52,unnamed_thm:66,unnatur:71,unnecessari:[8,17,57,62,66],unneed:[8,17,58],unop:5,unopspec:[5,17],unord:[3,17,57],unpack:17,unpredict:54,unprefix:3,unprocess:52,unprotect:[17,57],unprov:[17,43,58],unproven:[52,58,66],unqualifi:[17,35,55,71],unquot:[17,53,55],unquoted_str:53,unread:[17,59],unrealist:24,unreli:17,unresolv:[9,13,17,57,58,60,64,67],unrespons:17,unsaf:[2,17,55,66],unsafe_:17,unsafe_type_of:17,unsafecoerc:17,unsatisfi:[5,60],unselect:58,unset:[4,5,12,14,17,24,25,34,35,37,38,42,44,46,51,54,55,57,59,66,67,71],unshelv:[17,43,66],unsign:[5,17,36],unsolv:[9,17,43,66],unsound:[17,34],unspecifi:[4,14,17,43,55,62,67],unstabl:[14,17],unsuit:8,unsupport:[17,29,35,38,52,59],untermin:71,until:[13,14,17,24,26,31,32,34,40,52,54,55,57,60,64,66,67,72],untouch:[17,41],untyp:[10,17,25,55,71],unus:[17,25,53,58,71],unusu:17,unwant:17,up:[3,8,13,17,24,25,26,31,34,35,38,42,43,52,53,54,55,57,58,64,66,67,71,75],upcom:17,updat:[4,8,15,17,24,36,37,46,52,53,58,59,67,71],upfront:53,upgrad:[15,17,25],upon:[5,11,36,43,51],upper:[10,14,17,39,44,52],upper_bound_thm:17,uppercas:[29,55],upstream:[17,53],upward:[17,24],url:[17,27,52,75,77],us:[2,3,5,6,7,8,9,10,11,12,13,17,24,26,27,28,29,30,31,32,33,34,36,39,40,41,42,45,55,57,59,60,61,62,63,65,72,73,74,75,77],usa:77,usabl:[2,17,24,38,52,66,67,71],usag:[17,24,25,27,51,53,54,58,60,64],usecamlp4:17,usefulli:17,useless:[13,14,17,24,25,37,46,60],uselessli:17,uselocaldef:17,usepackag:75,user:[4,5,6,7,8,9,11,12,13,14,17,25,29,32,33,34,35,36,37,39,42,43,44,45,46,51,52,53,54,55,57,58,59,61,62,64,65,66,67,71,72,73,74,75,76,77],usernam:52,usual:[3,8,9,12,17,25,26,27,28,30,34,35,37,40,43,44,46,52,53,54,55,57,58,59,60,62,64,66,67,71,74,75],utf8:[52,53,75],utf8x:75,utf:[17,52,75],util:[17,42,51,53],v1:[25,50,57],v2:[24,57],v3:[24,57],v4:24,v5:24,v6:24,v7:[17,24],v8:17,v:[2,3,7,8,11,12,14,17,24,26,27,34,35,37,42,44,46,51,52,53,54,55,57,58,59,67,71,75],v_0:11,v_1:[11,31],v_2:11,v_3:11,v_:[11,26],v_i:[11,31],v_m:31,vadim:17,val:[2,34,55,57],valentin:17,valid:[2,3,4,5,8,10,11,14,17,25,26,29,32,34,35,40,42,51,54,55,57,58,59,66,71,72],valu:[2,4,5,6,9,11,12,13,14,17,24,25,26,27,28,29,31,32,34,36,37,38,40,42,43,51,52,53,57,58,59,60,62,64,66,67,71,74],value_tact:[52,54,64],van:17,vanish:24,vari:[24,54,58,67,71],variabl:[2,3,4,5,6,7,8,9,10,12,13,14,17,24,25,26,27,28,29,31,32,34,35,37,38,39,40,41,42,45,53,54,57,58,59,60,62,64,67,71,72,75],varianc:[3,17],variant:[5,13,14,17,24,25,27,28,29,32,33,34,35,37,38,42,51,54,55,59,60,63,64,66,67,71,72],variat:[17,59,77],varieti:[17,24],variou:[3,16,17,24,25,27,28,29,34,44,51,52,53,55,57,58,59,60,64,66,71],varmap:5,varnam:37,varner:17,varref:55,vassor:17,vax:24,vbt98:[3,77],vcon:[17,67],vdash:[0,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],vdfile:17,ve:[17,52,53,66,67],vec:67,vec_ind:67,vec_rec:67,vec_rect:67,vec_sind:67,vector:[17,46,67,71],vector_ind:67,vector_rec:67,vector_rect:67,vector_scop:17,vector_sind:67,vectordef:17,vectornot:17,vectorspec:17,vener:17,verbatim:25,verbos:[13,17,42,51,59],veri:[2,8,9,11,13,17,24,25,27,29,34,42,46,52,53,54,55,57,58,59,60,62,64,66,67],verif:[3,24,25,32,66,67,77],verifi:[3,7,9,11,14,17,24,25,29,31,32,33,35,51,60,66],verlag:77,vermand:17,vernac:[17,24,51,53,71,75],vernac_control:71,vernacular:[17,24,35,38,59,63,75],version:[2,3,4,7,9,13,14,15,25,29,32,34,35,36,37,41,46,50,51,52,57,58,59,60,62,66,73,74,75,77],versu:67,vertic:[17,59,71],vfile:53,vi:53,via:[2,5,8,11,17,35,51,53,54,55,57,59,71,72],vicent:17,view:[2,11,17,25,26,29,32,34,39,41,52,55,60,66],vincent:17,vindum:17,vio2vo:17,vio:17,violat:[39,66],virtu:17,virtual:[17,24,32,53,64],vis01:[3,77],visibl:[6,17,24,38,52,57,60,66,71,75],visser:[3,77],visual:[17,51,52,54,66,71],vlad:72,vm:[10,17,58,59,64],vm_c:53,vm_cast_no_check:58,vm_comput:[5,17,25,32,36,51,58],vmbyteflag:17,vnil:67,vo:[8,17,24,25,53,59],vocabulari:25,vofil:53,vok:[17,51],volatil:[17,32,41,46],volum:[24,77],volunt:17,vote:24,vs:[13,17,25,26],vscoq:[8,17,51,53,66],vulner:17,w:[0,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],w_1:[26,31],w_i:26,w_m:[26,31],wa:[2,3,10,11,12,17,24,27,28,29,32,34,35,37,38,41,42,43,44,51,52,53,54,55,57,58,59,60,63,64,66,67,71,72],wai:[2,3,5,11,12,13,14,17,24,25,26,27,29,30,31,32,34,35,37,42,43,44,46,51,52,53,57,58,59,60,62,63,64,66,67,71,72,73,75],wait:[17,55,66],waitpid:17,walding:24,walk:[55,71],wall:64,wand:77,wang:17,want:[2,11,13,17,34,35,36,41,42,43,51,52,53,54,55,57,58,59,60,62,64,66,67,71,73,74],warn:[2,3,4,10,12,13,16,17,24,25,27,28,29,32,34,35,37,41,42,44,46,51,52,54,55,57,59,60,62,66,71,72],we:[2,3,4,5,9,11,12,13,14,16,17,24,26,27,28,29,30,31,33,34,35,38,39,40,42,44,45,46,51,52,53,54,55,57,58,59,60,64,66,67,71,72,75],weak:[5,17,25,27,35,55,64,67,71],weaken:[17,67],weaker:[3,17,24,60],weakli:64,web:[17,27,52,53],websit:[17,75,76],wedg:7,weegen:17,week:17,wei:24,weid:17,weight:17,weird:17,welcom:[17,54],well:[2,3,4,8,9,10,11,13,14,17,24,25,26,29,30,31,32,33,35,37,39,43,45,46,51,52,53,54,55,57,58,59,63,64,66,67,71,72,74,75],well_found:27,well_founded_ind:27,well_founded_induct:[17,27],wellfound:[9,17,27],wendl:17,weng:17,went:[17,54,55],wenzel:17,wer94:[31,77],were:[3,11,13,17,24,34,35,36,38,42,44,51,53,54,55,59,60,66,71,72,75],werner:[11,17,24,77],wev:[0,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],weval:35,wevt:[0,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],weyhrauch:24,wf:[0,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],wf_lex_exp:17,wf_nat:[2,17,24],wf_simul:17,wf_slexprod:17,wf_z:24,wfe:[0,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],wft:[0,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],wftwolin:[0,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],what:[2,3,5,10,13,16,17,24,25,27,29,33,34,35,41,42,46,51,53,54,55,57,59,60,64,66,67,71],whatev:[3,44,64,75],whelp:17,when:[2,3,4,5,6,7,8,9,10,11,12,13,14,15,17,24,25,27,28,29,30,32,34,35,36,37,38,39,40,41,42,43,45,51,52,53,54,55,58,59,60,62,64,66,67,71,72,74,75],whenev:[3,7,14,17,27,29,42,55,57,62,64,67,71],where:[2,3,4,5,6,7,8,9,10,11,12,13,14,17,24,26,27,29,30,34,35,36,37,38,40,41,42,43,44,46,51,52,53,54,55,57,58,59,60,62,64,66,67,71,72,75],wherea:[17,29,54,55,57,58,62,74],wherev:[31,53,54,67,71],whether:[2,3,9,10,12,13,14,17,29,34,35,41,44,51,52,53,54,55,57,59,62,64,66,71,75],which:[2,3,4,5,6,7,8,9,10,11,12,13,14,17,24,25,26,27,28,29,30,31,32,33,34,35,36,37,38,39,40,41,42,43,44,45,46,51,52,53,54,55,57,58,59,60,62,63,64,65,66,67,71,72,73,75],whichev:17,whilst:9,white:[17,57],whitequark:17,whitespac:[17,24,53,75],who:[17,24,54,57,59],whole:[2,3,9,11,17,29,40,46,51,52,53,55,57,59,71,75],whose:[2,3,4,5,11,13,14,17,24,26,27,30,31,33,34,35,37,39,41,42,44,46,53,54,55,57,58,59,60,64,67,71,75],why2:17,why3:17,why:[3,11,17,34,37,43,55],wide:[29,38,52,53,58],widget:24,width:[17,59,71],wiedemann:17,wiedijk:24,wiki:[17,64],wikipedia:64,wilcox:17,wild:[17,57],wildcard:[9,13,25,28],william:77,win:17,window:[8,17,24,51,52,53],winterhalt:[17,77],wire:[17,55],wish:[2,5,17,53],wit:[5,14,17,24,27,39,55,64],with_declar:[17,35],with_strategi:[17,64,71],with_uniform_flag:54,within:[5,17,24,28,29,31,33,35,37,38,41,42,44,51,52,54,55,58,59,60,64,66,71],without:[2,3,5,8,9,11,13,14,17,24,26,29,32,33,34,35,37,42,43,44,46,51,52,53,54,55,57,58,59,60,63,64,66,67,71,74,75,77],wizard:14,wlia:5,wlog:[17,25],wlog_stat:57,wlra:5,wlra_q:5,wml07:77,wnia:5,wnra:5,wojciech:17,wolf:17,won:[17,25,38,52,53,54,55,58,62,64,67,71,73],word:[4,14,17,27,30,42,51,52,53,55,58,66],work:[2,3,4,5,9,10,12,13,17,24,25,26,27,32,35,41,42,43,46,51,52,54,55,57,58,59,64,67,71,74,77],workaround:[53,54,55,60],worker:[8,17,52,54],workflow:17,workshop:[24,77],workspac:17,workstat:24,world:[12,17,24,55,57,77],wors:55,worst:[17,59],worth:57,would:[2,3,4,11,14,17,28,29,30,31,32,34,37,41,42,43,44,46,53,54,55,57,58,59,60,62,64,66,67,71,72,75],wpsatz:5,wrap:[9,12,13,17,36,38,53],wrapper:[17,53,67,71,72],write:[3,4,8,11,13,14,17,24,25,26,27,29,31,32,33,34,38,39,43,51,53,54,55,57,58,59,63,66,67,71,73,75],writer:[17,29,55],written:[2,3,5,11,13,17,24,26,28,29,34,35,36,37,42,43,44,46,52,53,54,55,57,59,64,71,73,74],wrong:[2,3,17,24,44,51,54,66,72],wrongli:[17,46],wrongplu:34,wrote:[11,17,24],wrt:[17,24],ws:[0,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],wse:[0,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],wsl:52,wso:5,wt:[0,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],wte:[0,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],wteg:[0,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],wtm:[0,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],www:[17,24,25,27,50,75,77],x0:[3,13,17,37,43,44,54,66,71],x1:[3,9,13,17,27,42,54,57,59,60,72],x1p:36,x2:[3,27,42,59,60,72],x3:[27,71,72],x3p1:71,x3p2:71,x:[0,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],x_1:[7,26,34,35],x_:[7,34],x_j:34,x_k:[26,34],x_m:34,x_n:7,xa:57,xarg:17,xavier:[17,77],xb:57,xcolor:75,xdg:[17,53],xdg_config_hom:[17,51,52],xdg_data_dir:[17,51],xdg_data_hom:[17,51,53],xi:17,xia:17,xl:57,xlia:5,xlra:5,xmailserv:77,xml:[17,24],xn:[3,9,17,57],xnia:5,xnra:5,xo:17,xor:17,xorb:[17,27,59,62],xorb_comm:59,xp:17,xpsatz:5,xs:[58,64,67],xso:5,xx:17,xxx:14,xxx_scope:17,xxy:11,xyz:17,xz:11,y0:[3,13,43],y13:66,y1:[13,27,42,46,59],y2:[27,42,59],y3:27,y:[2,3,4,5,9,11,12,13,14,17,24,26,27,28,31,34,35,36,37,38,40,41,42,43,44,46,52,54,55,57,58,59,60,62,64,66,67,71,77],y_1:[34,38],y_:34,y_gt1:57,y_j:34,y_lt2:57,y_lt3:57,y_m:34,y_n:38,yale:17,yang:17,yann:[17,24],yannick:17,yao:17,ybertot:17,ye:[4,9,11,14,17,29,34,37,42,51,53,59,67],year:[17,24],yellow:[17,52],yet:[2,17,42,43,46,51,52,54,55,57,58,60,66,71,72],yice:17,yield:[4,11,17,24,31,46,54,55,58,67,71],yishuai:17,ym:57,ymmv:17,yojson:53,yop:24,york:77,yoshihiro:17,you:[2,3,4,7,8,10,11,13,14,15,16,17,24,25,27,29,32,34,35,37,41,43,44,46,51,52,53,54,55,57,58,59,60,62,64,66,67,71,72,73,74,75],your:[2,3,8,11,14,15,17,25,29,51,52,54,55,57,58,59,60,62,66,71,73,74,75],ype:77,ys:[46,58,67],ystem:77,yusuk:17,yve:[17,24,72],yx:11,yyy_scop:17,yz:11,z0:[11,17,71],z2nat:17,z3:17,z:[3,5,7,11,13,14,17,24,26,27,28,29,34,35,37,40,41,42,44,54,55,57,58,59,60,64,66,67,71],z_div_mod_eq:17,z_div_mod_eq_ful:17,z_le_gt_dec:17,z_lt_induct:17,z_lt_le_dec:17,z_scope:[5,11,17,27,66,71],za:[17,71],zaliva:17,zar:17,zarith:[5,11,17,24,27,29,53,57,60,66],zarith_aux:17,zarith_bas:17,zarith_base_modul:17,zarithr:11,zbinari:17,zbitwis:17,zchines:24,zcomplement:[17,24],zdigit:17,zdiv:17,zdiv_eucl_po:17,zdiv_fact:17,zdiveucl:17,zeimer:17,zeldovich:17,zenon:17,zero:[3,7,11,17,26,27,37,42,46,53,54,55,58,59,60,64],zeroon:[0,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],zeta:[17,24,31,55,64],zeuclid:17,zfc:24,zgt_square_simpl:17,zhong:77,zifi:[17,25],zify_convert_to_euclidean_division_equations_flag:5,zify_plugin:[11,27,29,36,54,55,57,60,66],zify_post_hook:[5,17],zify_pre_hook:[5,17],zifybool:[5,17],zifyclass:[5,17,57],zifycomparison:5,zifyinst:5,zifyint63:17,zifyn:[5,17],zifynat:[5,17],zifypow:17,zifysint63:5,zifyuint63:5,ziliani:[17,77],zim19:[74,77],zimmerman:[17,24],zimmermann:[17,77],zinc:[17,64,77],zine:77,zle:17,zle_0_plu:17,zle_mult_simpl:17,zle_zmult_pos_right:17,zle_zmult_right2:17,zlogarithm:[17,24],zlt_gt_succ:17,zlt_square_simpl:17,zlt_succ_gt:17,zmax:17,zmin:17,zminmax:17,zmisc:17,zmod:17,zmod_mod:17,zmod_neg_bound:17,zmod_pos_bound:17,zmodulo:17,zmult:24,zmult_1_n:17,zmult_assoc:17,zmult_assoc_l:17,zmult_comm:11,zmult_le_compat_r:17,zmult_minus_distr:17,zmult_on:17,zmult_zminus_distr_l:17,zmult_zminus_distr_r:17,zn2z:17,znatpair:17,znumtheori:17,zodiv:17,zplu:17,zplus_assoc:17,zplus_assoc_l:17,zplus_comm:17,zpo:17,zpower:[17,24],zpred:17,zsgn:24,zsqrt_compat:17,zulip:[17,52,54],zwanenburg:24,zx:11,zy:11,zyuzin:17},titles:["<no title>","<no title>","Program extraction","Generalized rewriting","Implicit Coercions","Micromega: solvers for arithmetic goals over ordered rings","Program derivation","Nsatz: a solver for equalities in integral domains","Asynchronous and Parallel Proof Processing","Program","User-defined rewrite rules","ring and field: solvers for polynomial and rational equations","SProp (proof irrelevant propositions)","Typeclasses","Polymorphic Universes","History and recent changes","Indexes","Recent changes","Attribute index","Command index","Errors and warnings index","Flags, options and tables index","Tactic index","General index","Early history of Coq","Introduction and Contents","Typing rules","The Coq library","Functions and assumptions","Basic notions and conventions","Coinductive types and corecursive functions","Conversion rules","Definitions","Core language","Inductive types and recursive functions","The Module System","Primitive objects","Record types","Sections","Sorts","Variants and the match construct","Setting properties of a function's arguments","Canonical Structures","Existential variables","Implicit arguments","Language extensions","Extended pattern matching","<no title>","<no title>","<no title>","<no title>","The Rocq Prover commands","CoqIDE","Building Rocq Projects","Ltac","Ltac2","<no title>","The SSReflect proof language","Tactics","Commands","Programmable proof search","Automatic solvers and programmable tactics","Solvers for logic and equality","Creating new tactics","Reasoning with equalities","Basic proof writing","Proof mode","Reasoning with inductive types","<no title>","Glossary index","<no title>","Syntax extensions and notation scopes","Functional induction","Libraries and plugins","Writing Rocq libraries and plugins","Documenting Rocq files with coqdoc","Command-line and graphical tools","Bibliography"],titleterms:{"0":[17,24],"0beta":17,"1":[17,24,37,67],"10":17,"11":17,"12":17,"13":17,"14":17,"15":17,"16":17,"17":17,"18":17,"19":17,"1beta":17,"1gamma":17,"2":[17,24,37,67],"20":17,"3":[17,24,71],"4":[17,24],"4beta":17,"4beta2":17,"5":[17,24],"5beta1":17,"5beta2":17,"5beta3":17,"5pl1":17,"5pl2":17,"5pl3":17,"6":[17,24],"6beta1":17,"7":[17,24],"8":17,"9":17,"\u03b1":31,"\u03b2":31,"\u03b4":31,"\u03b6":31,"\u03b7":31,"\u03b9":31,"abstract":[57,66],"boolean":[46,54,57],"byte":36,"case":[5,24,40,52,57,58,67],"catch":[54,55],"class":[3,4,37,55,71],"default":[41,46],"do":[11,54],"float":[27,36],"function":[4,28,30,34,41,44,54,60,72],"long":24,"new":[3,11,17,24,35,53,57,63],"short":5,"static":55,"switch":[55,57],"try":54,A:[2,14,35,58,67],In:55,Is:11,No:53,One:57,The:[11,26,27,34,35,44,51,53,57,71,75],_coqproject:53,abbrevi:[55,57,71],about:[7,46,71],access:37,ackermann:60,acknowledg:57,activ:4,ad:[3,11,52],addit:[2,57,60],advanc:[57,72],algorithm:64,alia:74,alias:46,altern:[41,54],alwai:64,ambigu:3,an:[35,57,59,67],analysi:67,annot:8,anonym:[37,57],antiquot:55,api:55,appendix:25,appli:[43,57,58,64,67],applic:[4,28,44,54,58],ar:[57,66],argument:[2,37,41,44,46,53,57,67,71],arithmet:[5,27],ariti:34,arrai:36,ask:9,assert:32,assert_fail:54,assert_succe:54,assign:57,associ:71,assumpt:[28,57],asynchron:[8,52],attribut:[4,17,18,29,35,38],autom:60,automat:[8,11,34,41,43,44,61,67],avail:4,avoid:2,axiom:2,b:58,backtrac:54,backtrack:[54,55,59],backward:[3,58],base:36,basic:[12,27,29,52,53,54,57,65,71],batch:51,beta1:17,beta2:17,beta3:17,beta:31,between:[2,55,59,66],bibliographi:77,bidirection:41,bind:[13,41,52,55,58,71],binder:[3,28,44,57,71],block:[8,57],bookkeep:57,both:71,bound:71,brace:66,branch:[54,57],breakpoint:52,buffer:52,build:[13,53],built:55,bullet:[57,66],calcul:66,calculu:26,call:[52,55],can:43,canon:42,cast:32,casual:44,caveat:[8,30],cell:55,chain:57,chang:[15,17,24,55],charact:52,check:54,checker:51,classic:58,claus:[37,46,58],clear:57,co:30,code:2,coercion:[4,46,71],cofix:30,coinduct:30,combin:[44,58,67],command:[3,13,17,19,24,35,51,52,57,59,66,67,71,75,76],comment:53,common:[53,58],compact:42,comparison:[54,55],compat:[10,17,37,55,57,74],compil:[17,51,52,53,59],complex:71,compon:55,compound:58,comput:[53,54,64],conclus:59,concret:[11,24],condit:[34,54,57],configur:53,conflict:2,confluenc:10,congruenc:57,connect:27,constant:[3,37,59,71],constraint:[14,66],construct:[12,24,26,34,37,40,54,59],constructor:[34,67],content:25,context:[3,13,54,55,57,58],contextu:[44,57],continu:[3,41,44],contradict:58,contravari:3,contribut:[2,24,27],control:[9,35,44,46,54,57,58,59,64,66],convent:[29,46],convers:[14,31,64],convert:31,coq:[24,27,52],coq_makefil:53,coqc:[51,53],coqchk:51,coqdep:53,coqdoc:75,coqid:[17,52],coqmakefil:53,coqrc:51,coqtop:51,core:33,corecurs:30,correct:34,count:54,covari:3,creat:[35,37,43,60,63],cumul:14,curli:66,custom:[51,52,71],cut:[5,54],cycl:66,databas:60,datatyp:27,deactiv:44,deal:11,debug:[12,54,55,59],debugg:[52,54],decid:[54,67],decis:5,declar:[3,13,38,41,42,44,55,57,66,67],defect:[54,57],defin:[10,34,35,37,54,55,60],definit:[3,9,12,14,30,32,34,37,40,46,54,55,57,64,71],delai:[55,66],delta:31,demonstr:14,depend:[17,46,53,58,59,67],deprec:[3,74],deriv:[6,42,67],descript:5,design:55,destruct:67,destructor:34,destructur:[46,57],detail:[2,17,24,53],detect:54,diff:66,differ:[2,44,66],disabl:71,disambigu:59,discharg:57,discrimin:67,discuss:11,disjunct:46,displai:[4,43,44,52,59,71],divis:2,document:[29,53,75],doe:[11,46],doesn:64,domain:7,dune:53,dynam:55,e:43,eappli:43,earli:24,eauto:13,edit:52,effect:[41,55],effici:24,elabor:9,element:[54,58],elim:57,elimin:[2,46,57],embed:53,emphasi:75,enabl:[3,66,71],encod:[12,52],end:[34,38],enter:66,entri:[57,71],environ:[51,59],equal:[7,9,27,62,64,67],equat:[11,57],equival:[57,58],error:[8,20,54,55],escap:75,essenti:29,eta:10,euclidean:2,eval:[54,64],evalu:[54,55],even:67,exact:57,exactly_onc:54,exampl:[2,3,4,5,6,11,14,17,26,27,28,29,30,31,34,35,37,38,40,41,42,43,44,46,51,52,53,54,55,57,58,59,60,62,64,66,67,71,72,74,75],except:55,execut:54,exist:[2,24,35],existenti:[43,57],exit:66,expans:[31,46],explicit:[14,43,44,57],explicitli:44,expos:59,express:[46,54,55,71],extend:[46,57],extens:[3,24,45,46,57,71],extra:[2,59],extract:[2,17,24],factor:[46,71],fail:[46,54,57],failur:54,famili:57,fast:[59,64],fatal:55,ffi:2,field:[11,35,37],file:[51,52,53,59,74,75],filenam:[2,53],fill:54,first:[3,34,46,54,57],fix:[31,34],fixpoint:[9,34],flag:[17,21,29,59],flow:[54,57,58],focus:[54,66],fold:64,fold_right:64,follow:44,foral:28,forbidden:53,forest:67,form:34,forward:58,found:27,frequent:9,fresh:54,from:[35,44,55],full:59,fun:28,function_scop:71,functor:35,gallina:57,gener:[2,3,4,11,14,23,29,44,54,55,57,67,71,72],get:[54,57],give:44,given:34,global:[14,54,71],glossari:69,goal:[5,11,54,55,57,58,66,67],grammar:[24,53],graph:4,graphic:76,guard:54,hand:46,have:[54,57],helper:67,hidden:46,hide:75,hierarchi:[13,42],high:5,higher:10,hint:[41,57,59,60],histor:24,histori:[11,15,24],hole:[10,54],horror:2,how:[11,66],html:75,hyperlink:75,hypothes:[54,55,58,59,66],hypothesi:[54,58],ident:[4,54],identifi:[59,71],idtac:54,implicit:[4,41,44,46,60,71],implicits_alt:41,impred:26,includ:58,incompat:[3,17],indent:57,index:[16,18,19,20,21,22,23,34,57,69],induct:[2,26,34,40,46,67,71,72],infer:[17,43,44],infix:71,inform:[66,71],infrastructur:17,inherit:[4,71],inlin:[2,59],innermost:3,input:52,insert:44,insid:[53,54,75],instal:53,instanc:[13,43],integ:[5,27,36,71],integr:7,interact:[8,35,44,51,54,55,57],interdepend:53,interfac:51,intern:59,interpret:[57,71],intro:[57,58],introduc:74,introduct:[3,25,57],intuitionist:54,invers:67,inversion_sigma:67,invoc:58,involv:[46,71],io:55,irrefut:46,irrelev:[12,31],is_cofix:54,is_fix:54,is_proj:54,isomorph:54,issu:[12,17,57],item:[35,57],iter:57,j:53,kei:52,kernel:17,keyword:[58,59],kind:44,knowledg:44,languag:[2,17,24,25,33,45,55,57],larger:67,late:53,latex:[53,75],launch:51,law:10,layer:55,lazy_match:55,lazymatch:54,least:54,left:67,leibniz:64,lemma:[9,27,66],let:[24,32,46,54,57],level:[5,10,29,30,32,34,55],lexic:29,lia:5,librari:[17,24,27,51,53,59,60,71,73,74],licit:57,limit:67,line:[17,51,75,76],linear:5,liner:57,list:[27,54,55,75],load:[51,53,59],local:[14,29,35,38,46,53,54,57,58,60,71],locat:[59,71],lock:57,logic:[27,53,54,60,62],loop:54,low:55,lower:34,lra:5,ltac1:55,ltac2:[17,55],ltac:[17,54,55],maccarthi:60,machin:59,macro:54,main:24,mainten:66,make:54,man:53,manag:[52,58,66],manipul:54,manual:[17,41,44],map:11,match:[31,34,37,40,46,54,55,57],materi:75,maxim:44,mechan:57,memori:66,meta:55,metavari:57,micromega:5,minim:14,miscellan:[17,24],ml:[2,55],mode:[8,44,52,55,57,66],modifi:53,modul:[4,35,53],monomorph:14,more:7,morphism:3,move:[57,58],multi:57,multi_match:55,multimatch:54,multipl:[37,41,46,53,54,55,57],museum:2,must:46,mutabl:55,mutual:34,n:67,name:[24,35,37,54,66],nat:[27,29],nativ:[17,53],native_comput:[53,64],natur:[54,55,60,67],neg:34,nest:[34,46],nia:5,non:[5,12,34,44,54,55,58,67,71],noncumul:14,nonreflex:3,nonsymmetr:3,notat:[17,27,42,54,55,59,71],notion:29,novelti:24,nra:5,nsatz:7,number:[27,54,60,71],numgoal:54,object:[34,36,46,74],oblig:9,ocaml:59,occurr:[34,57,58,67],odd:67,old:17,omit:35,onc:54,opam:53,opaqu:13,open:71,oper:59,optim:[2,54],option:[2,17,21,29,51,66,75],or_and_intropattern:67,order:[5,10,58],orient:58,other:[17,44,66],outermost:3,over:[5,9,55,57],overflow:29,overload:42,overview:[53,55],own:53,packag:53,page:53,parallel:8,paramet:[35,46,51,57],parameter:[13,34,71],parametr:[3,46,57],pars:[24,44,55,71],part:[59,75],partial:58,path:[53,59],pattern:[10,44,46,54,55,57,58,59,71],peano:27,perform:[53,58],permut:54,phrase:53,plane:5,plugin:[73,74],polymorph:[10,14,34,57],polynomi:11,posit:34,positivstellensatz:5,potenti:17,pre:5,preced:71,precompil:53,predefin:71,predic:[46,57,67],prefer:52,prelud:27,premis:[58,67],present:[4,14],preserv:10,pretti:[43,44,46,75],primit:[27,36,37,59,71],principl:[67,72,75],print:[3,4,14,37,43,44,46,54,55,59,71,75],privat:40,procedur:5,process:[5,8,54],produc:51,product:58,profil:[51,54,55],program:[2,6,9,27,55,60],programm:[60,61],progress:54,project:[37,53],proof:[5,8,12,14,25,31,32,46,54,57,58,60,65,66],prop:34,properti:[41,54,71],proposit:[12,27,54],prove:[54,66,67],prover:[25,51,53],provid:[3,46],psatz:5,qualifi:35,quantifi:27,queri:[52,59],question:9,quit:59,quot:53,quotat:55,radix:71,ration:[5,11],real:[5,17,27],realiz:2,reason:[58,64,67],recent:[15,17],record:[4,37],recurr:57,recurs:[27,30,34,55,71,72],redex:57,reduct:[24,31,34,37,55,59,64],refer:[17,54,59],reflect:57,refut:5,regist:59,registr:59,relat:3,remark:57,renam:41,reorder:[54,66],repeat:54,repetit:57,request:[59,66],reserv:[58,71],resili:8,resolut:[43,44,57],reus:37,revers:[4,44,54,55,64],revgoal:66,rewrit:[3,10,57,64,67],right:[46,67],ring:[5,11],rocq:[2,25,51,53,57,60,71,74,75],root:[24,53],rule:[10,26,31,34,38,57,64,71,75],run:[52,54],s:[2,27,41,67],same:[46,53],save:52,scheme:[67,72],scheme_typ:67,scope:[35,41,71],script:[51,52],search:[59,60],searchpattern:59,searchrewrit:59,second:[34,46,54,58],section:[4,13,14,38,66,75],select:57,selector:[54,57],semant:55,separ:66,sequenc:54,set:[2,13,26,29,37,41,57,58,60,66],setoid:[3,64],setup:53,share:35,shelv:66,shelve_unifi:66,shortcut:57,show:[66,75],side:[11,46],simpl:[28,31,34,35,55,64,71],simple_bind:58,simplif:57,simultan:71,singl:[51,54],soft:54,solv:[9,43,54,66],solver:[5,7,11,61,62],some:[2,27,35],sort:[14,34,39],sourc:[17,75],special:[57,58],specif:[17,25,27],specifi:14,split:[5,53],sprop:12,ssreflect:[17,57],stack:[29,52],standard:[17,24,27,55,57,60,71],start:[51,57],state:66,statu:59,step:[57,66],strategi:[3,46,64],strict:[12,34,44,55],strictli:34,string:[27,36,71],structur:[11,42,57],style:75,sub:35,subgoal:66,subpattern:46,subrel:3,subset:53,substitut:54,substructur:13,subterm:[43,46],subtyp:[26,44],succe:54,success:54,suff:57,suggest:8,summari:[13,17,24,35,38],superclass:13,support:[10,29,52],survei:27,swap:66,symbol:[10,52,54],synopsi:57,syntact:[9,54,55],syntax:[3,10,17,24,29,44,46,54,55,57,71],system:[2,35],t:64,tabl:[21,29],tactic:[3,5,11,17,22,24,27,43,54,55,57,58,60,61,63,64,67,71,72,74],target:[2,53],templat:[34,52],term:[26,54,55,64,71],termin:[10,12,57],test:[53,54],theorem:58,theori:34,thi:11,time:[51,53,54],time_constr:54,timeout:54,tool:[17,24,76],top:[30,32,34],toplevel:54,trace:54,trail:44,transit:55,transpar:13,tree:67,trigger:74,tryif:54,two:[35,54],type:[2,3,4,10,17,26,28,30,32,34,35,37,38,40,44,46,54,55,57,59,67,71],type_scop:71,type_term:54,typeclass:[13,57],uip:12,under:[3,57],understand:46,undo:64,unfold:[3,41,64],unicod:52,unif:[14,58,66],uninstal:53,univers:[10,14],unlock:57,unreleas:17,unset:29,until:58,untyp:54,unus:46,up:51,upgrad:53,us:[4,14,25,35,37,38,43,44,46,51,52,53,54,58,64,66,67,71],usag:[3,11,57,66,75],useless:2,user:[2,3,10,24,27],valu:[3,46,54,55],variabl:[11,43,44,46,51,52,55,66],varianc:14,variant:[40,46,57,58],variou:67,verbatim:75,version:[17,24,53],view:[5,57],vm_comput:64,vo:51,vocabulari:29,vs:[43,55,57],wai:[54,55],warn:[20,53,74],weak:14,well:[27,34],what:11,when:[44,46,57],wildcard:[46,57],wlog:57,work:[11,53,66],write:[46,65,74],your:53,zifi:5}}) \ No newline at end of file diff --git a/master/stdlib/Stdlib.Arith.Arith_base.html b/master/stdlib/Stdlib.Arith.Arith_base.html index 88a0392348..833a3d6f7d 100644 --- a/master/stdlib/Stdlib.Arith.Arith_base.html +++ b/master/stdlib/Stdlib.Arith.Arith_base.html @@ -58,7 +58,7 @@

Library Stdlib.Arith.Arith_base

-

arith hint database

+

arith hint database

@@ -80,7 +80,7 @@

Library Stdlib.Arith.Arith_base

-

lt and le

+

lt and le

diff --git a/master/stdlib/Stdlib.Arith.EqNat.html b/master/stdlib/Stdlib.Arith.EqNat.html index 40054aed99..ee8540cadf 100644 --- a/master/stdlib/Stdlib.Arith.EqNat.html +++ b/master/stdlib/Stdlib.Arith.EqNat.html @@ -56,7 +56,7 @@

Library Stdlib.Arith.EqNat

Equality on natural numbers
-

Propositional equality

+

Propositional equality

diff --git a/master/stdlib/Stdlib.Arith.PeanoNat.html b/master/stdlib/Stdlib.Arith.PeanoNat.html index 415fa2a6cc..ffbc839d00 100644 --- a/master/stdlib/Stdlib.Arith.PeanoNat.html +++ b/master/stdlib/Stdlib.Arith.PeanoNat.html @@ -149,7 +149,7 @@

Library Stdlib.Arith.PeanoNat

-

Remaining constants not defined in Stdlib.Init.Nat

+

Remaining constants not defined in Stdlib.Init.Nat

@@ -167,7 +167,7 @@

Library Stdlib.Arith.PeanoNat

-

Basic specifications : pred add sub mul

+

Basic specifications : pred add sub mul

@@ -209,7 +209,7 @@

Library Stdlib.Arith.PeanoNat

-

Boolean comparisons

+

Boolean comparisons

@@ -241,7 +241,7 @@

Library Stdlib.Arith.PeanoNat

-

Decidability of equality over nat.

+

Decidability of equality over nat.

@@ -253,7 +253,7 @@

Library Stdlib.Arith.PeanoNat

-

Ternary comparison

+

Ternary comparison

@@ -282,7 +282,7 @@

Library Stdlib.Arith.PeanoNat

-

Minimum, maximum

+

Minimum, maximum

@@ -332,7 +332,7 @@

Library Stdlib.Arith.PeanoNat

-

Power

+

Power

@@ -350,7 +350,7 @@

Library Stdlib.Arith.PeanoNat

-

Square

+

Square

@@ -362,7 +362,7 @@

Library Stdlib.Arith.PeanoNat

-

Parity

+

Parity

@@ -406,7 +406,7 @@

Library Stdlib.Arith.PeanoNat

-

Division

+

Division

@@ -435,7 +435,7 @@

Library Stdlib.Arith.PeanoNat

-

Square root

+

Square root

@@ -459,7 +459,7 @@

Library Stdlib.Arith.PeanoNat

-

Logarithm

+

Logarithm

@@ -481,7 +481,7 @@

Library Stdlib.Arith.PeanoNat

-

Properties of iter

+

Properties of iter

@@ -533,7 +533,7 @@

Library Stdlib.Arith.PeanoNat

-

Gcd

+

Gcd

@@ -561,7 +561,7 @@

Library Stdlib.Arith.PeanoNat

-

Bitwise operations

+

Bitwise operations

diff --git a/master/stdlib/Stdlib.Bool.Bool.html b/master/stdlib/Stdlib.Bool.Bool.html index f30219dadd..583a5f0e45 100644 --- a/master/stdlib/Stdlib.Bool.Bool.html +++ b/master/stdlib/Stdlib.Bool.Bool.html @@ -90,7 +90,7 @@

Library Stdlib.Bool.Bool

-

Decidability

+

Decidability

@@ -102,7 +102,7 @@

Library Stdlib.Bool.Bool

-

Discrimination

+

Discrimination

@@ -138,7 +138,7 @@

Library Stdlib.Bool.Bool

-

Order on booleans

+

Order on booleans

@@ -180,7 +180,7 @@

Library Stdlib.Bool.Bool

-

Equality

+

Equality

@@ -223,7 +223,7 @@

Library Stdlib.Bool.Bool

-

A synonym of if on bool

+

A synonym of if on bool

@@ -242,7 +242,7 @@

Library Stdlib.Bool.Bool

-

De Morgan laws

+

De Morgan laws

@@ -257,7 +257,7 @@

Library Stdlib.Bool.Bool

-

Properties of negb

+

Properties of negb

@@ -299,7 +299,7 @@

Library Stdlib.Bool.Bool

-

Properties of orb

+

Properties of orb

@@ -427,7 +427,7 @@

Library Stdlib.Bool.Bool

-

Properties of andb

+

Properties of andb

@@ -544,7 +544,7 @@

Library Stdlib.Bool.Bool

-

Properties mixing andb and orb

+

Properties mixing andb and orb

@@ -594,7 +594,7 @@

Library Stdlib.Bool.Bool

-

Properties of implb

+

Properties of implb

@@ -648,7 +648,7 @@

Library Stdlib.Bool.Bool

-

Properties of xorb

+

Properties of xorb

@@ -810,7 +810,7 @@

Library Stdlib.Bool.Bool

-

Reflection of bool into Prop

+

Reflection of bool into Prop

@@ -924,7 +924,7 @@

Library Stdlib.Bool.Bool

-

Alternative versions of andb and orb

+

Alternative versions of andb and orb

with lazy behavior (for vm_compute)
@@ -952,7 +952,7 @@

Library Stdlib.Bool.Bool

-

Reflect: a specialized inductive type for

+

Reflect: a specialized inductive type for

relating propositions and booleans, as popularized by the Ssreflect library. diff --git a/master/stdlib/Stdlib.Bool.BoolOrder.html b/master/stdlib/Stdlib.Bool.BoolOrder.html index cd3c5ac48f..9e5f9a6506 100644 --- a/master/stdlib/Stdlib.Bool.BoolOrder.html +++ b/master/stdlib/Stdlib.Bool.BoolOrder.html @@ -66,7 +66,7 @@

Library Stdlib.Bool.BoolOrder

-

Order le

+

Order le

@@ -92,7 +92,7 @@

Library Stdlib.Bool.BoolOrder

-

Strict order lt

+

Strict order lt

@@ -127,7 +127,7 @@

Library Stdlib.Bool.BoolOrder

-

Order structures

+

Order structures

diff --git a/master/stdlib/Stdlib.Classes.CEquivalence.html b/master/stdlib/Stdlib.Classes.CEquivalence.html index d2fb159734..8b0b543f11 100644 --- a/master/stdlib/Stdlib.Classes.CEquivalence.html +++ b/master/stdlib/Stdlib.Classes.CEquivalence.html @@ -49,7 +49,7 @@

Library Stdlib.Classes.CEquivalence

-

Typeclass-based setoids. Definitions on Equivalence.

+

Typeclass-based setoids. Definitions on Equivalence.

diff --git a/master/stdlib/Stdlib.Classes.CMorphisms.html b/master/stdlib/Stdlib.Classes.CMorphisms.html index 1f25a72cd5..06b4e78587 100644 --- a/master/stdlib/Stdlib.Classes.CMorphisms.html +++ b/master/stdlib/Stdlib.Classes.CMorphisms.html @@ -49,7 +49,7 @@

Library Stdlib.Classes.CMorphisms

-

Typeclass-based morphism definition and standard, minimal instances

+

Typeclass-based morphism definition and standard, minimal instances

@@ -78,7 +78,7 @@

Library Stdlib.Classes.CMorphisms

-

Morphisms.

+

Morphisms.

diff --git a/master/stdlib/Stdlib.Classes.CRelationClasses.html b/master/stdlib/Stdlib.Classes.CRelationClasses.html index f16e08a915..f978d2a5b7 100644 --- a/master/stdlib/Stdlib.Classes.CRelationClasses.html +++ b/master/stdlib/Stdlib.Classes.CRelationClasses.html @@ -49,7 +49,7 @@

Library Stdlib.Classes.CRelationClasses

-

Typeclass-based relations, tactics and standard instances

+

Typeclass-based relations, tactics and standard instances

@@ -454,7 +454,7 @@

Library Stdlib.Classes.CRelationClasses

We can already dualize all these properties.
-

Standard instances.

+

Standard instances.

@@ -607,7 +607,7 @@

Library Stdlib.Classes.CRelationClasses

-

Partial Order.

+

Partial Order.

A partial order is a preorder which is additionally antisymmetric. We give an equivalent definition, up-to an equivalence crelation diff --git a/master/stdlib/Stdlib.Classes.DecidableClass.html b/master/stdlib/Stdlib.Classes.DecidableClass.html index 760efce841..1f82fc6681 100644 --- a/master/stdlib/Stdlib.Classes.DecidableClass.html +++ b/master/stdlib/Stdlib.Classes.DecidableClass.html @@ -49,7 +49,7 @@

Library Stdlib.Classes.DecidableClass

-

A typeclass to ease the handling of decidable properties.

+

A typeclass to ease the handling of decidable properties.

diff --git a/master/stdlib/Stdlib.Classes.EquivDec.html b/master/stdlib/Stdlib.Classes.EquivDec.html index c1ca13f0ed..e2ac23ebb5 100644 --- a/master/stdlib/Stdlib.Classes.EquivDec.html +++ b/master/stdlib/Stdlib.Classes.EquivDec.html @@ -49,7 +49,7 @@

Library Stdlib.Classes.EquivDec

-

Decidable equivalences.

+

Decidable equivalences.

diff --git a/master/stdlib/Stdlib.Classes.Equivalence.html b/master/stdlib/Stdlib.Classes.Equivalence.html index b21f0acb5c..ff63304ce7 100644 --- a/master/stdlib/Stdlib.Classes.Equivalence.html +++ b/master/stdlib/Stdlib.Classes.Equivalence.html @@ -49,7 +49,7 @@

Library Stdlib.Classes.Equivalence

-

Typeclass-based setoids. Definitions on Equivalence.

+

Typeclass-based setoids. Definitions on Equivalence.

diff --git a/master/stdlib/Stdlib.Classes.Init.html b/master/stdlib/Stdlib.Classes.Init.html index 828b5e5bbc..dfcfd54348 100644 --- a/master/stdlib/Stdlib.Classes.Init.html +++ b/master/stdlib/Stdlib.Classes.Init.html @@ -49,7 +49,7 @@

Library Stdlib.Classes.Init

-

Initialization code for typeclasses, setting up the default tactic

+

Initialization code for typeclasses, setting up the default tactic

for instance search. diff --git a/master/stdlib/Stdlib.Classes.Morphisms.html b/master/stdlib/Stdlib.Classes.Morphisms.html index e4e170ce82..259c10485e 100644 --- a/master/stdlib/Stdlib.Classes.Morphisms.html +++ b/master/stdlib/Stdlib.Classes.Morphisms.html @@ -49,7 +49,7 @@

Library Stdlib.Classes.Morphisms

-

Typeclass-based morphism definition and standard, minimal instances

+

Typeclass-based morphism definition and standard, minimal instances

@@ -74,7 +74,7 @@

Library Stdlib.Classes.Morphisms

-

Morphisms.

+

Morphisms.

diff --git a/master/stdlib/Stdlib.Classes.Morphisms_Prop.html b/master/stdlib/Stdlib.Classes.Morphisms_Prop.html index b98d0bc213..2c059d1a2b 100644 --- a/master/stdlib/Stdlib.Classes.Morphisms_Prop.html +++ b/master/stdlib/Stdlib.Classes.Morphisms_Prop.html @@ -49,7 +49,7 @@

Library Stdlib.Classes.Morphisms_Prop

-

Proper instances for propositional connectives.

+

Proper instances for propositional connectives.

diff --git a/master/stdlib/Stdlib.Classes.Morphisms_Relations.html b/master/stdlib/Stdlib.Classes.Morphisms_Relations.html index dd6c4e27e8..224b1ea831 100644 --- a/master/stdlib/Stdlib.Classes.Morphisms_Relations.html +++ b/master/stdlib/Stdlib.Classes.Morphisms_Relations.html @@ -49,7 +49,7 @@

Library Stdlib.Classes.Morphisms_Relations

-

Morphism instances for relations.

+

Morphism instances for relations.

diff --git a/master/stdlib/Stdlib.Classes.RelationClasses.html b/master/stdlib/Stdlib.Classes.RelationClasses.html index 014e9bac2c..4c1aa3f8c9 100644 --- a/master/stdlib/Stdlib.Classes.RelationClasses.html +++ b/master/stdlib/Stdlib.Classes.RelationClasses.html @@ -49,7 +49,7 @@

Library Stdlib.Classes.RelationClasses

-

Typeclass-based relations, tactics and standard instances

+

Typeclass-based relations, tactics and standard instances

@@ -480,7 +480,7 @@

Library Stdlib.Classes.RelationClasses

We can already dualize all these properties.
-

Standard instances.

+

Standard instances.

@@ -847,7 +847,7 @@

Library Stdlib.Classes.RelationClasses

-

Partial Order.

+

Partial Order.

A partial order is a preorder which is additionally antisymmetric. We give an equivalent definition, up-to an equivalence relation diff --git a/master/stdlib/Stdlib.Classes.RelationPairs.html b/master/stdlib/Stdlib.Classes.RelationPairs.html index a8d8da293d..680db6cf8d 100644 --- a/master/stdlib/Stdlib.Classes.RelationPairs.html +++ b/master/stdlib/Stdlib.Classes.RelationPairs.html @@ -49,7 +49,7 @@

Library Stdlib.Classes.RelationPairs

-

Relations over pairs

+

Relations over pairs

diff --git a/master/stdlib/Stdlib.Classes.SetoidClass.html b/master/stdlib/Stdlib.Classes.SetoidClass.html index 8f153b0376..e966eeb7df 100644 --- a/master/stdlib/Stdlib.Classes.SetoidClass.html +++ b/master/stdlib/Stdlib.Classes.SetoidClass.html @@ -49,7 +49,7 @@

Library Stdlib.Classes.SetoidClass

-

Typeclass-based setoids, tactics and standard instances.

+

Typeclass-based setoids, tactics and standard instances.

diff --git a/master/stdlib/Stdlib.Classes.SetoidDec.html b/master/stdlib/Stdlib.Classes.SetoidDec.html index ac2b8dd578..3be8a7fefd 100644 --- a/master/stdlib/Stdlib.Classes.SetoidDec.html +++ b/master/stdlib/Stdlib.Classes.SetoidDec.html @@ -49,7 +49,7 @@

Library Stdlib.Classes.SetoidDec

-

Decidable setoid equality theory.

+

Decidable setoid equality theory.

diff --git a/master/stdlib/Stdlib.Classes.SetoidTactics.html b/master/stdlib/Stdlib.Classes.SetoidTactics.html index 57c34c0375..355600fa53 100644 --- a/master/stdlib/Stdlib.Classes.SetoidTactics.html +++ b/master/stdlib/Stdlib.Classes.SetoidTactics.html @@ -49,7 +49,7 @@

Library Stdlib.Classes.SetoidTactics

-

Tactics for typeclass-based setoids.

+

Tactics for typeclass-based setoids.

diff --git a/master/stdlib/Stdlib.FSets.FMapAVL.html b/master/stdlib/Stdlib.FSets.FMapAVL.html index 8a5f806701..a5f22df368 100644 --- a/master/stdlib/Stdlib.FSets.FMapAVL.html +++ b/master/stdlib/Stdlib.FSets.FMapAVL.html @@ -51,7 +51,7 @@

Library Stdlib.FSets.FMapAVL

-

FMapAVL

+

FMapAVL

@@ -88,7 +88,7 @@

Library Stdlib.FSets.FMapAVL

-

The Raw functor

+

The Raw functor

@@ -114,11 +114,11 @@

Library Stdlib.FSets.FMapAVL

-

Trees

+

Trees

-

Trees

+

Trees

@@ -150,7 +150,7 @@

Library Stdlib.FSets.FMapAVL

-

Basic functions on trees: height and cardinal

+

Basic functions on trees: height and cardinal

@@ -173,7 +173,7 @@

Library Stdlib.FSets.FMapAVL

-

Empty Map

+

Empty Map

@@ -185,7 +185,7 @@

Library Stdlib.FSets.FMapAVL

-

Emptyness test

+

Emptyness test

@@ -197,7 +197,7 @@

Library Stdlib.FSets.FMapAVL

-

Membership

+

Membership

@@ -232,7 +232,7 @@

Library Stdlib.FSets.FMapAVL

-

Helper functions

+

Helper functions

@@ -295,7 +295,7 @@

Library Stdlib.FSets.FMapAVL

-

Insertion

+

Insertion

@@ -316,7 +316,7 @@

Library Stdlib.FSets.FMapAVL

-

Extraction of minimum binding

+

Extraction of minimum binding

@@ -341,7 +341,7 @@

Library Stdlib.FSets.FMapAVL

-

Merging two trees

+

Merging two trees

@@ -367,7 +367,7 @@

Library Stdlib.FSets.FMapAVL

-

Deletion

+

Deletion

@@ -387,7 +387,7 @@

Library Stdlib.FSets.FMapAVL

-

join

+

join

@@ -416,7 +416,7 @@

Library Stdlib.FSets.FMapAVL

-

Splitting

+

Splitting

@@ -456,7 +456,7 @@

Library Stdlib.FSets.FMapAVL

-

Concatenation

+

Concatenation

@@ -480,7 +480,7 @@

Library Stdlib.FSets.FMapAVL

-

Elements

+

Elements

@@ -511,7 +511,7 @@

Library Stdlib.FSets.FMapAVL

-

Fold

+

Fold

@@ -527,7 +527,7 @@

Library Stdlib.FSets.FMapAVL

-

Comparison

+

Comparison

@@ -539,7 +539,7 @@

Library Stdlib.FSets.FMapAVL

-

Enumeration of the elements of a tree

+

Enumeration of the elements of a tree

@@ -638,7 +638,7 @@

Library Stdlib.FSets.FMapAVL

-

Map

+

Map

@@ -663,7 +663,7 @@

Library Stdlib.FSets.FMapAVL

-

Map with removal

+

Map with removal

@@ -684,7 +684,7 @@

Library Stdlib.FSets.FMapAVL

-

Optimized map2

+

Optimized map2

@@ -740,7 +740,7 @@

Library Stdlib.FSets.FMapAVL

-

Map2

+

Map2

@@ -770,7 +770,7 @@

Library Stdlib.FSets.FMapAVL

-

Invariants

+

Invariants

@@ -783,7 +783,7 @@

Library Stdlib.FSets.FMapAVL

-

Occurrence in a tree

+

Occurrence in a tree

@@ -813,7 +813,7 @@

Library Stdlib.FSets.FMapAVL

-

Binary search trees

+

Binary search trees

@@ -847,7 +847,7 @@

Library Stdlib.FSets.FMapAVL

-

Correctness proofs, isolated in a sub-module

+

Correctness proofs, isolated in a sub-module

@@ -1139,7 +1139,7 @@

Library Stdlib.FSets.FMapAVL

-

Automation and dedicated tactics.

+

Automation and dedicated tactics.

@@ -1250,7 +1250,7 @@

Library Stdlib.FSets.FMapAVL

-

Basic results about MapsTo, In, lt_tree, gt_tree, height

+

Basic results about MapsTo, In, lt_tree, gt_tree, height

@@ -1354,7 +1354,7 @@

Library Stdlib.FSets.FMapAVL

-

Empty map

+

Empty map

@@ -1372,7 +1372,7 @@

Library Stdlib.FSets.FMapAVL

-

Emptyness test

+

Emptyness test

@@ -1387,7 +1387,7 @@

Library Stdlib.FSets.FMapAVL

-

Membership

+

Membership

@@ -1441,7 +1441,7 @@

Library Stdlib.FSets.FMapAVL

-

Helper functions

+

Helper functions

@@ -1481,7 +1481,7 @@

Library Stdlib.FSets.FMapAVL

-

Insertion

+

Insertion

@@ -1515,7 +1515,7 @@

Library Stdlib.FSets.FMapAVL

-

Extraction of minimum binding

+

Extraction of minimum binding

@@ -1558,7 +1558,7 @@

Library Stdlib.FSets.FMapAVL

-

Merging two trees

+

Merging two trees

@@ -1580,7 +1580,7 @@

Library Stdlib.FSets.FMapAVL

-

Deletion

+

Deletion

@@ -1607,7 +1607,7 @@

Library Stdlib.FSets.FMapAVL

-

join

+

join

@@ -1631,7 +1631,7 @@

Library Stdlib.FSets.FMapAVL

-

split

+

split

@@ -1670,7 +1670,7 @@

Library Stdlib.FSets.FMapAVL

-

Concatenation

+

Concatenation

@@ -1696,7 +1696,7 @@

Library Stdlib.FSets.FMapAVL

-

Elements

+

Elements

@@ -1750,7 +1750,7 @@

Library Stdlib.FSets.FMapAVL

-

Fold

+

Fold

@@ -1778,7 +1778,7 @@

Library Stdlib.FSets.FMapAVL

-

Comparison

+

Comparison

@@ -2005,7 +2005,7 @@

Library Stdlib.FSets.FMapAVL

-

Encapsulation

+

Encapsulation

diff --git a/master/stdlib/Stdlib.FSets.FMapFacts.html b/master/stdlib/Stdlib.FSets.FMapFacts.html index 31eece9de8..26c672dbde 100644 --- a/master/stdlib/Stdlib.FSets.FMapFacts.html +++ b/master/stdlib/Stdlib.FSets.FMapFacts.html @@ -49,7 +49,7 @@

Library Stdlib.FSets.FMapFacts

-

Finite maps library

+

Finite maps library

@@ -76,7 +76,7 @@

Library Stdlib.FSets.FMapFacts

-

Facts about weak maps

+

Facts about weak maps

@@ -103,7 +103,7 @@

Library Stdlib.FSets.FMapFacts

-

Specifications written using equivalences

+

Specifications written using equivalences

@@ -260,7 +260,7 @@

Library Stdlib.FSets.FMapFacts

-

Specifications written using boolean predicates

+

Specifications written using boolean predicates

@@ -399,7 +399,7 @@

Library Stdlib.FSets.FMapFacts

-

Relations between Equal, Equiv and Equivb.

+

Relations between Equal, Equiv and Equivb.

@@ -461,7 +461,7 @@

Library Stdlib.FSets.FMapFacts

-

Equal is a setoid equality.

+

Equal is a setoid equality.

@@ -545,7 +545,7 @@

Library Stdlib.FSets.FMapFacts

-

Same facts for self-contained weak sets and for full maps

+

Same facts for self-contained weak sets and for full maps

@@ -558,7 +558,7 @@

Library Stdlib.FSets.FMapFacts

-

Additional Properties for weak maps

+

Additional Properties for weak maps

@@ -618,7 +618,7 @@

Library Stdlib.FSets.FMapFacts

-

Elements

+

Elements

@@ -633,7 +633,7 @@

Library Stdlib.FSets.FMapFacts

-

Conversions between maps and association lists.

+

Conversions between maps and association lists.

@@ -670,7 +670,7 @@

Library Stdlib.FSets.FMapFacts

-

Fold

+

Fold

@@ -686,7 +686,7 @@

Library Stdlib.FSets.FMapFacts

-

Induction principles about fold contributed by S. Lescuyer

+

Induction principles about fold contributed by S. Lescuyer

@@ -799,7 +799,7 @@

Library Stdlib.FSets.FMapFacts

-

Additional properties of fold

+

Additional properties of fold

@@ -894,7 +894,7 @@

Library Stdlib.FSets.FMapFacts

-

Cardinal

+

Cardinal

@@ -940,7 +940,7 @@

Library Stdlib.FSets.FMapFacts

-

Additional notions over maps

+

Additional notions over maps

@@ -958,7 +958,7 @@

Library Stdlib.FSets.FMapFacts

-

Emulation of some functions lacking in the interface

+

Emulation of some functions lacking in the interface

@@ -1185,7 +1185,7 @@

Library Stdlib.FSets.FMapFacts

-

Same Properties for self-contained weak maps and for full maps

+

Same Properties for self-contained weak maps and for full maps

@@ -1198,7 +1198,7 @@

Library Stdlib.FSets.FMapFacts

-

Properties specific to maps with ordered keys

+

Properties specific to maps with ordered keys

diff --git a/master/stdlib/Stdlib.FSets.FMapFullAVL.html b/master/stdlib/Stdlib.FSets.FMapFullAVL.html index 3b2a781053..1d3080aa35 100644 --- a/master/stdlib/Stdlib.FSets.FMapFullAVL.html +++ b/master/stdlib/Stdlib.FSets.FMapFullAVL.html @@ -51,7 +51,7 @@

Library Stdlib.FSets.FMapFullAVL

-

FMapFullAVL

+

FMapFullAVL

@@ -120,7 +120,7 @@

Library Stdlib.FSets.FMapFullAVL

-

AVL trees

+

AVL trees

@@ -144,7 +144,7 @@

Library Stdlib.FSets.FMapFullAVL

-

Automation and dedicated tactics about avl.

+

Automation and dedicated tactics about avl.

@@ -182,7 +182,7 @@

Library Stdlib.FSets.FMapFullAVL

-

Basic results about avl, height

+

Basic results about avl, height

@@ -210,7 +210,7 @@

Library Stdlib.FSets.FMapFullAVL

-

Empty map

+

Empty map

@@ -222,7 +222,7 @@

Library Stdlib.FSets.FMapFullAVL

-

Helper functions

+

Helper functions

@@ -262,7 +262,7 @@

Library Stdlib.FSets.FMapFullAVL

-

Insertion

+

Insertion

@@ -280,7 +280,7 @@

Library Stdlib.FSets.FMapFullAVL

-

Extraction of minimum binding

+

Extraction of minimum binding

@@ -298,7 +298,7 @@

Library Stdlib.FSets.FMapFullAVL

-

Merging two trees

+

Merging two trees

@@ -317,7 +317,7 @@

Library Stdlib.FSets.FMapFullAVL

-

Deletion

+

Deletion

@@ -335,7 +335,7 @@

Library Stdlib.FSets.FMapFullAVL

-

Join

+

Join

@@ -454,7 +454,7 @@

Library Stdlib.FSets.FMapFullAVL

-

Encapsulation

+

Encapsulation

@@ -653,7 +653,7 @@

Library Stdlib.FSets.FMapFullAVL

-

As comparison function, we propose here a non-structural

+

As comparison function, we propose here a non-structural

version faithful to the code of Ocaml's Map library, instead of the structural version of FMapAVL diff --git a/master/stdlib/Stdlib.FSets.FMapInterface.html b/master/stdlib/Stdlib.FSets.FMapInterface.html index bbe3f611c5..272a468f94 100644 --- a/master/stdlib/Stdlib.FSets.FMapInterface.html +++ b/master/stdlib/Stdlib.FSets.FMapInterface.html @@ -49,7 +49,7 @@

Library Stdlib.FSets.FMapInterface

-

Finite map library

+

Finite map library

@@ -135,7 +135,7 @@

Library Stdlib.FSets.FMapInterface

-

Weak signature for maps

+

Weak signature for maps

@@ -556,7 +556,7 @@

Library Stdlib.FSets.FMapInterface

-

Static signature for Weak Maps

+

Static signature for Weak Maps

@@ -575,7 +575,7 @@

Library Stdlib.FSets.FMapInterface

-

Maps on ordered keys, functorial signature

+

Maps on ordered keys, functorial signature

@@ -602,7 +602,7 @@

Library Stdlib.FSets.FMapInterface

-

Maps on ordered keys, self-contained signature

+

Maps on ordered keys, self-contained signature

@@ -617,7 +617,7 @@

Library Stdlib.FSets.FMapInterface

-

Maps with ordering both on keys and datas

+

Maps with ordering both on keys and datas

diff --git a/master/stdlib/Stdlib.FSets.FMapList.html b/master/stdlib/Stdlib.FSets.FMapList.html index beb80d06d9..9297513b24 100644 --- a/master/stdlib/Stdlib.FSets.FMapList.html +++ b/master/stdlib/Stdlib.FSets.FMapList.html @@ -49,7 +49,7 @@

Library Stdlib.FSets.FMapList

-

Finite map library

+

Finite map library

@@ -93,7 +93,7 @@

Library Stdlib.FSets.FMapList

-

empty

+

empty

@@ -116,7 +116,7 @@

Library Stdlib.FSets.FMapList

-

is_empty

+

is_empty

@@ -134,7 +134,7 @@

Library Stdlib.FSets.FMapList

-

mem

+

mem

@@ -161,7 +161,7 @@

Library Stdlib.FSets.FMapList

-

find

+

find

@@ -188,7 +188,7 @@

Library Stdlib.FSets.FMapList

-

add

+

add

@@ -229,7 +229,7 @@

Library Stdlib.FSets.FMapList

-

remove

+

remove

@@ -270,7 +270,7 @@

Library Stdlib.FSets.FMapList

-

elements

+

elements

@@ -296,7 +296,7 @@

Library Stdlib.FSets.FMapList

-

fold

+

fold

@@ -316,7 +316,7 @@

Library Stdlib.FSets.FMapList

-

equal

+

equal

@@ -366,7 +366,7 @@

Library Stdlib.FSets.FMapList

-

map and mapi

+

map and mapi

@@ -459,7 +459,7 @@

Library Stdlib.FSets.FMapList

-

map2

+

map2

diff --git a/master/stdlib/Stdlib.FSets.FMapPositive.html b/master/stdlib/Stdlib.FSets.FMapPositive.html index ec0a9e745e..e6a76444ee 100644 --- a/master/stdlib/Stdlib.FSets.FMapPositive.html +++ b/master/stdlib/Stdlib.FSets.FMapPositive.html @@ -49,7 +49,7 @@

Library Stdlib.FSets.FMapPositive

-

FMapPositive : an implementation of FMapInterface for positive keys.

+

FMapPositive : an implementation of FMapInterface for positive keys.

diff --git a/master/stdlib/Stdlib.FSets.FMapWeakList.html b/master/stdlib/Stdlib.FSets.FMapWeakList.html index 48a59cbf5b..ee4078de48 100644 --- a/master/stdlib/Stdlib.FSets.FMapWeakList.html +++ b/master/stdlib/Stdlib.FSets.FMapWeakList.html @@ -49,7 +49,7 @@

Library Stdlib.FSets.FMapWeakList

-

Finite map library

+

Finite map library

@@ -91,7 +91,7 @@

Library Stdlib.FSets.FMapWeakList

-

empty

+

empty

@@ -116,7 +116,7 @@

Library Stdlib.FSets.FMapWeakList

-

is_empty

+

is_empty

@@ -134,7 +134,7 @@

Library Stdlib.FSets.FMapWeakList

-

mem

+

mem

@@ -156,7 +156,7 @@

Library Stdlib.FSets.FMapWeakList

-

find

+

find

@@ -185,7 +185,7 @@

Library Stdlib.FSets.FMapWeakList

-

add

+

add

@@ -229,7 +229,7 @@

Library Stdlib.FSets.FMapWeakList

-

remove

+

remove

@@ -263,7 +263,7 @@

Library Stdlib.FSets.FMapWeakList

-

elements

+

elements

@@ -284,7 +284,7 @@

Library Stdlib.FSets.FMapWeakList

-

fold

+

fold

@@ -304,7 +304,7 @@

Library Stdlib.FSets.FMapWeakList

-

equal

+

equal

@@ -365,7 +365,7 @@

Library Stdlib.FSets.FMapWeakList

-

map and mapi

+

map and mapi

diff --git a/master/stdlib/Stdlib.FSets.FSetAVL.html b/master/stdlib/Stdlib.FSets.FSetAVL.html index 3b01b23b89..13d0c0ec92 100644 --- a/master/stdlib/Stdlib.FSets.FSetAVL.html +++ b/master/stdlib/Stdlib.FSets.FSetAVL.html @@ -49,7 +49,7 @@

Library Stdlib.FSets.FSetAVL

-

FSetAVL : Implementation of FSetInterface via AVL trees

+

FSetAVL : Implementation of FSetInterface via AVL trees

diff --git a/master/stdlib/Stdlib.FSets.FSetBridge.html b/master/stdlib/Stdlib.FSets.FSetBridge.html index 77bb5e5793..4a09946258 100644 --- a/master/stdlib/Stdlib.FSets.FSetBridge.html +++ b/master/stdlib/Stdlib.FSets.FSetBridge.html @@ -49,7 +49,7 @@

Library Stdlib.FSets.FSetBridge

-

Finite sets library

+

Finite sets library

@@ -66,7 +66,7 @@

Library Stdlib.FSets.FSetBridge

-

From non-dependent signature S to dependent signature Sdep.

+

From non-dependent signature S to dependent signature Sdep.

@@ -244,7 +244,7 @@

Library Stdlib.FSets.FSetBridge

-

From dependent signature Sdep to non-dependent signature S.

+

From dependent signature Sdep to non-dependent signature S.

diff --git a/master/stdlib/Stdlib.FSets.FSetCompat.html b/master/stdlib/Stdlib.FSets.FSetCompat.html index 5b66121a8e..aa2c889a5b 100644 --- a/master/stdlib/Stdlib.FSets.FSetCompat.html +++ b/master/stdlib/Stdlib.FSets.FSetCompat.html @@ -49,7 +49,7 @@

Library Stdlib.FSets.FSetCompat

-

Compatibility functors between FSetInterface and MSetInterface.

+

Compatibility functors between FSetInterface and MSetInterface.

@@ -65,7 +65,7 @@

Library Stdlib.FSets.FSetCompat

-

From new Weak Sets to old ones

+

From new Weak Sets to old ones

@@ -228,7 +228,7 @@

Library Stdlib.FSets.FSetCompat

-

From new Sets to new ones

+

From new Sets to new ones

@@ -286,7 +286,7 @@

Library Stdlib.FSets.FSetCompat

-

From old Weak Sets to new ones.

+

From old Weak Sets to new ones.

@@ -429,7 +429,7 @@

Library Stdlib.FSets.FSetCompat

-

From old Sets to new ones.

+

From old Sets to new ones.

diff --git a/master/stdlib/Stdlib.FSets.FSetDecide.html b/master/stdlib/Stdlib.FSets.FSetDecide.html index 6abb2d8387..53187565c8 100644 --- a/master/stdlib/Stdlib.FSets.FSetDecide.html +++ b/master/stdlib/Stdlib.FSets.FSetDecide.html @@ -75,7 +75,7 @@

Library Stdlib.FSets.FSetDecide

-

Overview

+

Overview

This functor defines the tactic fsetdec, which will solve any valid goal of the form @@ -181,7 +181,7 @@

Library Stdlib.FSets.FSetDecide

-

Facts and Tactics for Propositional Logic

+

Facts and Tactics for Propositional Logic

These lemmas and tactics are in a module so that they do not affect the namespace if you import the enclosing @@ -196,18 +196,18 @@

Library Stdlib.FSets.FSetDecide

-

Lemmas and Tactics About Decidable Propositions

+

Lemmas and Tactics About Decidable Propositions

-

Propositional Equivalences Involving Negation

+

Propositional Equivalences Involving Negation

These are all written with the unfolded form of negation, since I am not sure if setoid rewriting will always perform conversion.
-

Tactics for Negations

+

Tactics for Negations

@@ -458,7 +458,7 @@

Library Stdlib.FSets.FSetDecide

-

Auxiliary Tactics

+

Auxiliary Tactics

Again, these lemmas and tactics are in a module so that they do not affect the namespace if you import the @@ -471,7 +471,7 @@

Library Stdlib.FSets.FSetDecide

-

Generic Tactics

+

Generic Tactics

We begin by defining a few generic, useful tactics.
@@ -588,7 +588,7 @@

Library Stdlib.FSets.FSetDecide

-

Discarding Irrelevant Hypotheses

+

Discarding Irrelevant Hypotheses

We will want to clear the context of any non-FSet-related hypotheses in order to increase the @@ -668,7 +668,7 @@

Library Stdlib.FSets.FSetDecide

-

Turning Set Operators into Propositional Connectives

+

Turning Set Operators into Propositional Connectives

The lemmas from FSetFacts will be used to break down set operations into propositional formulas built over @@ -694,7 +694,7 @@

Library Stdlib.FSets.FSetDecide

-

Decidability of FSet Propositions

+

Decidability of FSet Propositions

@@ -729,7 +729,7 @@

Library Stdlib.FSets.FSetDecide

-

Normalizing Propositions About Equality

+

Normalizing Propositions About Equality

We have to deal with the fact that E.eq may be convertible with Coq's equality. Thus, we will find the @@ -812,7 +812,7 @@

Library Stdlib.FSets.FSetDecide

-

Considering Decidability of Base Propositions

+

Considering Decidability of Base Propositions

This tactic adds assertions about the decidability of E.eq and In to the context. This is necessary for @@ -861,7 +861,7 @@

Library Stdlib.FSets.FSetDecide

-

Handling Empty, Subset, and Equal

+

Handling Empty, Subset, and Equal

This tactic instantiates universally quantified hypotheses (which arise from the unfolding of Empty, @@ -909,7 +909,7 @@

Library Stdlib.FSets.FSetDecide

-

The Core fsetdec Auxiliary Tactics

+

The Core fsetdec Auxiliary Tactics

@@ -951,7 +951,7 @@

Library Stdlib.FSets.FSetDecide

-

The fsetdec Tactic

+

The fsetdec Tactic

Here is the top-level tactic (the only one intended for clients of this library). It's specification is given at @@ -1065,7 +1065,7 @@

Library Stdlib.FSets.FSetDecide

-

Examples

+

Examples

diff --git a/master/stdlib/Stdlib.FSets.FSetEqProperties.html b/master/stdlib/Stdlib.FSets.FSetEqProperties.html index bf21f71a9d..4c9d3ef159 100644 --- a/master/stdlib/Stdlib.FSets.FSetEqProperties.html +++ b/master/stdlib/Stdlib.FSets.FSetEqProperties.html @@ -49,7 +49,7 @@

Library Stdlib.FSets.FSetEqProperties

-

Finite sets library

+

Finite sets library

diff --git a/master/stdlib/Stdlib.FSets.FSetFacts.html b/master/stdlib/Stdlib.FSets.FSetFacts.html index fa4329f766..941ffc5a04 100644 --- a/master/stdlib/Stdlib.FSets.FSetFacts.html +++ b/master/stdlib/Stdlib.FSets.FSetFacts.html @@ -49,7 +49,7 @@

Library Stdlib.FSets.FSetFacts

-

Finite sets library

+

Finite sets library

@@ -85,7 +85,7 @@

Library Stdlib.FSets.FSetFacts

-

Specifications written using equivalences

+

Specifications written using equivalences

@@ -179,7 +179,7 @@

Library Stdlib.FSets.FSetFacts

-

Specifications written using boolean predicates

+

Specifications written using boolean predicates

@@ -243,7 +243,7 @@

Library Stdlib.FSets.FSetFacts

-

E.eq and Equal are setoid equalities

+

E.eq and Equal are setoid equalities

diff --git a/master/stdlib/Stdlib.FSets.FSetInterface.html b/master/stdlib/Stdlib.FSets.FSetInterface.html index 4e13fd7e47..1b54f6625f 100644 --- a/master/stdlib/Stdlib.FSets.FSetInterface.html +++ b/master/stdlib/Stdlib.FSets.FSetInterface.html @@ -49,7 +49,7 @@

Library Stdlib.FSets.FSetInterface

-

Finite set library

+

Finite set library

@@ -105,7 +105,7 @@

Library Stdlib.FSets.FSetInterface

-

Non-dependent signatures

+

Non-dependent signatures

@@ -114,7 +114,7 @@

Library Stdlib.FSets.FSetInterface

programs together with axioms
-

Functorial signature for weak sets

+

Functorial signature for weak sets

@@ -619,7 +619,7 @@

Library Stdlib.FSets.FSetInterface

-

Static signature for weak sets

+

Static signature for weak sets

@@ -639,7 +639,7 @@

Library Stdlib.FSets.FSetInterface

-

Functorial signature for sets on ordered elements

+

Functorial signature for sets on ordered elements

@@ -766,7 +766,7 @@

Library Stdlib.FSets.FSetInterface

-

Static signature for sets on ordered elements

+

Static signature for sets on ordered elements

@@ -786,7 +786,7 @@

Library Stdlib.FSets.FSetInterface

-

Some subtyping tests

+

Some subtyping tests

 WSfun ---> WS
@@ -803,7 +803,7 @@ 

Library Stdlib.FSets.FSetInterface

-

Dependent signature

+

Dependent signature

diff --git a/master/stdlib/Stdlib.FSets.FSetList.html b/master/stdlib/Stdlib.FSets.FSetList.html index 89a8ffe8a3..6ba5377d36 100644 --- a/master/stdlib/Stdlib.FSets.FSetList.html +++ b/master/stdlib/Stdlib.FSets.FSetList.html @@ -49,7 +49,7 @@

Library Stdlib.FSets.FSetList

-

Finite sets library

+

Finite sets library

diff --git a/master/stdlib/Stdlib.FSets.FSetProperties.html b/master/stdlib/Stdlib.FSets.FSetProperties.html index 74dc8f5195..7095152c70 100644 --- a/master/stdlib/Stdlib.FSets.FSetProperties.html +++ b/master/stdlib/Stdlib.FSets.FSetProperties.html @@ -49,7 +49,7 @@

Library Stdlib.FSets.FSetProperties

-

Finite sets library

+

Finite sets library

@@ -341,7 +341,7 @@

Library Stdlib.FSets.FSetProperties

-

Properties of elements

+

Properties of elements

@@ -356,7 +356,7 @@

Library Stdlib.FSets.FSetProperties

-

Conversions between lists and sets

+

Conversions between lists and sets

@@ -380,7 +380,7 @@

Library Stdlib.FSets.FSetProperties

-

Fold

+

Fold

@@ -408,7 +408,7 @@

Library Stdlib.FSets.FSetProperties

-

Induction principles for fold (contributed by S. Lescuyer)

+

Induction principles for fold (contributed by S. Lescuyer)

@@ -514,7 +514,7 @@

Library Stdlib.FSets.FSetProperties

-

Alternative (weaker) specifications for fold

+

Alternative (weaker) specifications for fold

@@ -586,7 +586,7 @@

Library Stdlib.FSets.FSetProperties

-

Fold is a morphism

+

Fold is a morphism

@@ -603,7 +603,7 @@

Library Stdlib.FSets.FSetProperties

-

Fold and other set operators

+

Fold and other set operators

@@ -655,11 +655,11 @@

Library Stdlib.FSets.FSetProperties

-

Cardinal

+

Cardinal

-

Characterization of cardinal in terms of fold

+

Characterization of cardinal in terms of fold

@@ -671,7 +671,7 @@

Library Stdlib.FSets.FSetProperties

-

Old specifications for cardinal.

+

Old specifications for cardinal.

@@ -694,7 +694,7 @@

Library Stdlib.FSets.FSetProperties

-

Cardinal and (non-)emptiness

+

Cardinal and (non-)emptiness

@@ -719,7 +719,7 @@

Library Stdlib.FSets.FSetProperties

-

Cardinal is a morphism

+

Cardinal is a morphism

@@ -738,7 +738,7 @@

Library Stdlib.FSets.FSetProperties

-

Cardinal and set operators

+

Cardinal and set operators

diff --git a/master/stdlib/Stdlib.FSets.FSetToFiniteSet.html b/master/stdlib/Stdlib.FSets.FSetToFiniteSet.html index 2628b39d3a..f9fc11d901 100644 --- a/master/stdlib/Stdlib.FSets.FSetToFiniteSet.html +++ b/master/stdlib/Stdlib.FSets.FSetToFiniteSet.html @@ -49,7 +49,7 @@

Library Stdlib.FSets.FSetToFiniteSet

-

Finite sets library : conversion to old Finite_sets

+

Finite sets library : conversion to old Finite_sets

@@ -62,7 +62,7 @@

Library Stdlib.FSets.FSetToFiniteSet

-

Going from FSets with usual Leibniz equality

+

Going from FSets with usual Leibniz equality

to the good old Ensembles and Finite_sets theory.
diff --git a/master/stdlib/Stdlib.FSets.FSetWeakList.html b/master/stdlib/Stdlib.FSets.FSetWeakList.html index bcc744919a..c95eb828fe 100644 --- a/master/stdlib/Stdlib.FSets.FSetWeakList.html +++ b/master/stdlib/Stdlib.FSets.FSetWeakList.html @@ -49,7 +49,7 @@

Library Stdlib.FSets.FSetWeakList

-

Finite sets library

+

Finite sets library

diff --git a/master/stdlib/Stdlib.Floats.FloatAxioms.html b/master/stdlib/Stdlib.Floats.FloatAxioms.html index c244c7b3d6..22f5ae6d31 100644 --- a/master/stdlib/Stdlib.Floats.FloatAxioms.html +++ b/master/stdlib/Stdlib.Floats.FloatAxioms.html @@ -52,7 +52,7 @@

Library Stdlib.Floats.FloatAxioms

-

Properties of the primitive operators for the Binary64 format

+

Properties of the primitive operators for the Binary64 format

diff --git a/master/stdlib/Stdlib.Floats.FloatLemmas.html b/master/stdlib/Stdlib.Floats.FloatLemmas.html index 3d30dcc741..07598bdb6d 100644 --- a/master/stdlib/Stdlib.Floats.FloatLemmas.html +++ b/master/stdlib/Stdlib.Floats.FloatLemmas.html @@ -53,7 +53,7 @@

Library Stdlib.Floats.FloatLemmas

-

Support results involving frexp and ldexp

+

Support results involving frexp and ldexp

diff --git a/master/stdlib/Stdlib.Floats.FloatOps.html b/master/stdlib/Stdlib.Floats.FloatOps.html index a929258538..f855a7e550 100644 --- a/master/stdlib/Stdlib.Floats.FloatOps.html +++ b/master/stdlib/Stdlib.Floats.FloatOps.html @@ -52,7 +52,7 @@

Library Stdlib.Floats.FloatOps

-

Derived operations and mapping between primitive floats and spec_floats

+

Derived operations and mapping between primitive floats and spec_floats

diff --git a/master/stdlib/Stdlib.Floats.PrimFloat.html b/master/stdlib/Stdlib.Floats.PrimFloat.html index 9ae95158fd..84709a65f3 100644 --- a/master/stdlib/Stdlib.Floats.PrimFloat.html +++ b/master/stdlib/Stdlib.Floats.PrimFloat.html @@ -52,7 +52,7 @@

Library Stdlib.Floats.PrimFloat

-

Definition of the interface for primitive floating-point arithmetic

+

Definition of the interface for primitive floating-point arithmetic

@@ -61,7 +61,7 @@

Library Stdlib.Floats.PrimFloat

IEEE 754-2008 standard.
-

Type definition for the co-domain of compare

+

Type definition for the co-domain of compare

@@ -77,7 +77,7 @@

Library Stdlib.Floats.PrimFloat

-

The main type

+

The main type

float: primitive type for Binary64 floating-point numbers.
@@ -95,7 +95,7 @@

Library Stdlib.Floats.PrimFloat

-

Syntax support

+

Syntax support

@@ -110,7 +110,7 @@

Library Stdlib.Floats.PrimFloat

-

Floating-point operators

+

Floating-point operators

@@ -185,7 +185,7 @@

Library Stdlib.Floats.PrimFloat

-

Conversions

+

Conversions

@@ -224,7 +224,7 @@

Library Stdlib.Floats.PrimFloat

-

Exponent manipulation functions

+

Exponent manipulation functions

frshiftexp: convert a float to fractional part in [0.5, 1.) and integer part.
@@ -244,7 +244,7 @@

Library Stdlib.Floats.PrimFloat

-

Predecesor/Successor functions

+

Predecesor/Successor functions

@@ -266,7 +266,7 @@

Library Stdlib.Floats.PrimFloat

-

Special values (needed for pretty-printing)

+

Special values (needed for pretty-printing)

@@ -283,7 +283,7 @@

Library Stdlib.Floats.PrimFloat

-

Other special values

+

Other special values

@@ -296,7 +296,7 @@

Library Stdlib.Floats.PrimFloat

-

Predicates and helper functions

+

Predicates and helper functions

diff --git a/master/stdlib/Stdlib.Floats.SpecFloat.html b/master/stdlib/Stdlib.Floats.SpecFloat.html index fa6c55fc20..bc0b4d6510 100644 --- a/master/stdlib/Stdlib.Floats.SpecFloat.html +++ b/master/stdlib/Stdlib.Floats.SpecFloat.html @@ -52,7 +52,7 @@

Library Stdlib.Floats.SpecFloat

-

Specification of floating-point arithmetic

+

Specification of floating-point arithmetic

@@ -61,7 +61,7 @@

Library Stdlib.Floats.SpecFloat

of the Flocq library (see http://flocq.gforge.inria.fr/)
-

Inductive specification of floating-point numbers

+

Inductive specification of floating-point numbers

@@ -79,7 +79,7 @@

Library Stdlib.Floats.SpecFloat

-

Parameterized definitions

+

Parameterized definitions

@@ -242,7 +242,7 @@

Library Stdlib.Floats.SpecFloat

-

Define operations

+

Define operations

diff --git a/master/stdlib/Stdlib.Init.Byte.html b/master/stdlib/Stdlib.Init.Byte.html index c5dbdb0538..655d20eb74 100644 --- a/master/stdlib/Stdlib.Init.Byte.html +++ b/master/stdlib/Stdlib.Init.Byte.html @@ -49,7 +49,7 @@

Library Stdlib.Init.Byte

-

Bytes

+

Bytes

diff --git a/master/stdlib/Stdlib.Init.Datatypes.html b/master/stdlib/Stdlib.Init.Datatypes.html index 171f2c2dab..8ed0316688 100644 --- a/master/stdlib/Stdlib.Init.Datatypes.html +++ b/master/stdlib/Stdlib.Init.Datatypes.html @@ -57,7 +57,7 @@

Library Stdlib.Init.Datatypes

-

Datatypes with zero and one element

+

Datatypes with zero and one element

@@ -91,7 +91,7 @@

Library Stdlib.Init.Datatypes

-

The boolean datatype

+

The boolean datatype

@@ -262,7 +262,7 @@

Library Stdlib.Init.Datatypes

-

Peano natural numbers

+

Peano natural numbers

@@ -297,7 +297,7 @@

Library Stdlib.Init.Datatypes

-

Container datatypes

+

Container datatypes

@@ -502,7 +502,7 @@

Library Stdlib.Init.Datatypes

-

The comparison datatype

+

The comparison datatype

@@ -620,7 +620,7 @@

Library Stdlib.Init.Datatypes

-

Misc Other Datatypes

+

Misc Other Datatypes

diff --git a/master/stdlib/Stdlib.Init.Decimal.html b/master/stdlib/Stdlib.Init.Decimal.html index cc19a807aa..2e7b616f96 100644 --- a/master/stdlib/Stdlib.Init.Decimal.html +++ b/master/stdlib/Stdlib.Init.Decimal.html @@ -49,7 +49,7 @@

Library Stdlib.Init.Decimal

-

Decimal numbers

+

Decimal numbers

diff --git a/master/stdlib/Stdlib.Init.Hexadecimal.html b/master/stdlib/Stdlib.Init.Hexadecimal.html index 1617033c6c..d496bf3f65 100644 --- a/master/stdlib/Stdlib.Init.Hexadecimal.html +++ b/master/stdlib/Stdlib.Init.Hexadecimal.html @@ -49,7 +49,7 @@

Library Stdlib.Init.Hexadecimal

-

Hexadecimal numbers

+

Hexadecimal numbers

diff --git a/master/stdlib/Stdlib.Init.Logic.html b/master/stdlib/Stdlib.Init.Logic.html index a112022ffd..782aec6b2b 100644 --- a/master/stdlib/Stdlib.Init.Logic.html +++ b/master/stdlib/Stdlib.Init.Logic.html @@ -59,7 +59,7 @@

Library Stdlib.Init.Logic

-

Propositional connectives

+

Propositional connectives

@@ -314,7 +314,7 @@

Library Stdlib.Init.Logic

-

First-order quantifiers

+

First-order quantifiers

@@ -467,7 +467,7 @@

Library Stdlib.Init.Logic

-

Equality

+

Equality

@@ -867,7 +867,7 @@

Library Stdlib.Init.Logic

-

Being inhabited

+

Being inhabited

diff --git a/master/stdlib/Stdlib.Init.Nat.html b/master/stdlib/Stdlib.Init.Nat.html index 120df3fcd9..3f18d6038d 100644 --- a/master/stdlib/Stdlib.Init.Nat.html +++ b/master/stdlib/Stdlib.Init.Nat.html @@ -54,7 +54,7 @@

Library Stdlib.Init.Nat

-

Peano natural numbers, definitions of operations

+

Peano natural numbers, definitions of operations

@@ -71,7 +71,7 @@

Library Stdlib.Init.Nat

-

Constants

+

Constants

@@ -90,7 +90,7 @@

Library Stdlib.Init.Nat

-

Basic operations

+

Basic operations

@@ -159,7 +159,7 @@

Library Stdlib.Init.Nat

-

Comparisons

+

Comparisons

@@ -205,7 +205,7 @@

Library Stdlib.Init.Nat

-

Minimum, maximum

+

Minimum, maximum

@@ -230,7 +230,7 @@

Library Stdlib.Init.Nat

-

Parity tests

+

Parity tests

@@ -250,7 +250,7 @@

Library Stdlib.Init.Nat

-

Power

+

Power

@@ -268,7 +268,7 @@

Library Stdlib.Init.Nat

-

Tail-recursive versions of add and mul

+

Tail-recursive versions of add and mul

@@ -302,7 +302,7 @@

Library Stdlib.Init.Nat

-

Conversion with a decimal representation for printing/parsing

+

Conversion with a decimal representation for printing/parsing

@@ -426,7 +426,7 @@

Library Stdlib.Init.Nat

-

Euclidean division

+

Euclidean division

@@ -469,7 +469,7 @@

Library Stdlib.Init.Nat

-

Greatest common divisor

+

Greatest common divisor

@@ -491,7 +491,7 @@

Library Stdlib.Init.Nat

-

Square

+

Square

@@ -503,7 +503,7 @@

Library Stdlib.Init.Nat

-

Square root

+

Square root

@@ -541,7 +541,7 @@

Library Stdlib.Init.Nat

-

Log2

+

Log2

diff --git a/master/stdlib/Stdlib.Init.Number.html b/master/stdlib/Stdlib.Init.Number.html index a965af976b..75b2b470d3 100644 --- a/master/stdlib/Stdlib.Init.Number.html +++ b/master/stdlib/Stdlib.Init.Number.html @@ -49,7 +49,7 @@

Library Stdlib.Init.Number

-

Decimal or Hexadecimal numbers

+

Decimal or Hexadecimal numbers

diff --git a/master/stdlib/Stdlib.Init.Tactics.html b/master/stdlib/Stdlib.Init.Tactics.html index cf9ca6fd2a..f3939c28ef 100644 --- a/master/stdlib/Stdlib.Init.Tactics.html +++ b/master/stdlib/Stdlib.Init.Tactics.html @@ -55,7 +55,7 @@

Library Stdlib.Init.Tactics

-

Useful tactics

+

Useful tactics

@@ -376,7 +376,7 @@

Library Stdlib.Init.Tactics

-

inversion_sigma

+

inversion_sigma

The built-in inversion will frequently leave equalities of dependent pairs. When the first type in the pair is an hProp or otherwise simplifies, inversion_sigma is useful; it will replace diff --git a/master/stdlib/Stdlib.Init.Tauto.html b/master/stdlib/Stdlib.Init.Tauto.html index d33b4bdf7e..cfa2336e8d 100644 --- a/master/stdlib/Stdlib.Init.Tauto.html +++ b/master/stdlib/Stdlib.Init.Tauto.html @@ -49,7 +49,7 @@

Library Stdlib.Init.Tauto

-

The tauto and intuition tactics

+

The tauto and intuition tactics

diff --git a/master/stdlib/Stdlib.Init.Wf.html b/master/stdlib/Stdlib.Init.Wf.html index 7139b9cc10..184dd25edf 100644 --- a/master/stdlib/Stdlib.Init.Wf.html +++ b/master/stdlib/Stdlib.Init.Wf.html @@ -49,7 +49,7 @@

Library Stdlib.Init.Wf

-

This module proves the validity of

+

This module proves the validity of

  • well-founded recursion (also known as course of values) diff --git a/master/stdlib/Stdlib.Lists.List.html b/master/stdlib/Stdlib.Lists.List.html index 3c6a2e1c3a..62d24970b6 100644 --- a/master/stdlib/Stdlib.Lists.List.html +++ b/master/stdlib/Stdlib.Lists.List.html @@ -56,7 +56,7 @@

    Library Stdlib.Lists.List

-

Basics: definition of polymorphic lists and some operations

+

Basics: definition of polymorphic lists and some operations

@@ -148,7 +148,7 @@

Library Stdlib.Lists.List

-

Generic facts

+

Generic facts

@@ -183,7 +183,7 @@

Library Stdlib.Lists.List

-

Head and tail

+

Head and tail

@@ -198,7 +198,7 @@

Library Stdlib.Lists.List

-

Facts about app

+

Facts about app

@@ -316,7 +316,7 @@

Library Stdlib.Lists.List

-

Facts about In

+

Facts about In

@@ -403,7 +403,7 @@

Library Stdlib.Lists.List

-

Operations on the elements of a list

+

Operations on the elements of a list

@@ -418,7 +418,7 @@

Library Stdlib.Lists.List

-

Nth element of a list

+

Nth element of a list

@@ -620,7 +620,7 @@

Library Stdlib.Lists.List

-

Last element of a list

+

Last element of a list

@@ -675,7 +675,7 @@

Library Stdlib.Lists.List

-

Remove

+

Remove

@@ -726,7 +726,7 @@

Library Stdlib.Lists.List

-

Counting occurrences of an element

+

Counting occurrences of an element

@@ -789,7 +789,7 @@

Library Stdlib.Lists.List

-

Manipulating whole lists

+

Manipulating whole lists

@@ -804,7 +804,7 @@

Library Stdlib.Lists.List

-

Reverse

+

Reverse

@@ -901,7 +901,7 @@

Library Stdlib.Lists.List

-

Concatenation

+

Concatenation

@@ -930,7 +930,7 @@

Library Stdlib.Lists.List

-

Decidable equality on lists

+

Decidable equality on lists

@@ -951,11 +951,11 @@

Library Stdlib.Lists.List

-

Applying functions to the elements of a list

+

Applying functions to the elements of a list

-

Map

+

Map

@@ -1046,7 +1046,7 @@

Library Stdlib.Lists.List

-

Flat Map

+

Flat Map

@@ -1228,7 +1228,7 @@

Library Stdlib.Lists.List

-

Boolean operations over lists

+

Boolean operations over lists

@@ -1395,7 +1395,7 @@

Library Stdlib.Lists.List

-

Further filtering facts

+

Further filtering facts

@@ -1489,7 +1489,7 @@

Library Stdlib.Lists.List

-

Operations on lists of pairs or lists of lists

+

Operations on lists of pairs or lists of lists

@@ -1621,11 +1621,11 @@

Library Stdlib.Lists.List

-

Miscellaneous operations on lists

+

Miscellaneous operations on lists

-

Length order of lists

+

Length order of lists

@@ -1669,7 +1669,7 @@

Library Stdlib.Lists.List

-

Set inclusion on list

+

Set inclusion on list

@@ -1759,7 +1759,7 @@

Library Stdlib.Lists.List

-

Cutting a list at some position

+

Cutting a list at some position

@@ -1938,7 +1938,7 @@

Library Stdlib.Lists.List

-

Combining pairs of lists of possibly-different lengths

+

Combining pairs of lists of possibly-different lengths

@@ -1970,7 +1970,7 @@

Library Stdlib.Lists.List

-

Predicate for List addition/removal (no need for decidability)

+

Predicate for List addition/removal (no need for decidability)

@@ -2014,7 +2014,7 @@

Library Stdlib.Lists.List

-

Lists without redundancy

+

Lists without redundancy

@@ -2166,7 +2166,7 @@

Library Stdlib.Lists.List

-

Sequence of natural numbers

+

Sequence of natural numbers

@@ -2233,7 +2233,7 @@

Library Stdlib.Lists.List

-

List comparison

+

List comparison

@@ -2379,7 +2379,7 @@

Library Stdlib.Lists.List

-

Existential and universal predicates over lists

+

Existential and universal predicates over lists

@@ -2911,7 +2911,7 @@

Library Stdlib.Lists.List

-

Inversion of predicates over lists based on head symbol

+

Inversion of predicates over lists based on head symbol

@@ -2939,7 +2939,7 @@

Library Stdlib.Lists.List

-

Exporting hints and tactics

+

Exporting hints and tactics

diff --git a/master/stdlib/Stdlib.Lists.SetoidList.html b/master/stdlib/Stdlib.Lists.SetoidList.html index 93a849993c..c28af4cc8b 100644 --- a/master/stdlib/Stdlib.Lists.SetoidList.html +++ b/master/stdlib/Stdlib.Lists.SetoidList.html @@ -53,7 +53,7 @@

Library Stdlib.Lists.SetoidList

-

Logical relations over lists with respect to a setoid equality

+

Logical relations over lists with respect to a setoid equality

or ordering.
diff --git a/master/stdlib/Stdlib.Lists.StreamMemo.html b/master/stdlib/Stdlib.Lists.StreamMemo.html index 33888adffb..4b622656bd 100644 --- a/master/stdlib/Stdlib.Lists.StreamMemo.html +++ b/master/stdlib/Stdlib.Lists.StreamMemo.html @@ -53,7 +53,7 @@

Library Stdlib.Lists.StreamMemo

-

Memoization

+

Memoization

diff --git a/master/stdlib/Stdlib.Logic.ChoiceFacts.html b/master/stdlib/Stdlib.Logic.ChoiceFacts.html index 41332aa540..6a07001a8f 100644 --- a/master/stdlib/Stdlib.Logic.ChoiceFacts.html +++ b/master/stdlib/Stdlib.Logic.ChoiceFacts.html @@ -50,7 +50,7 @@

Library Stdlib.Logic.ChoiceFacts

Some facts and definitions concerning choice and description in - intuitionistic logic.

References:

+ intuitionistic logic.

References:

@@ -89,7 +89,7 @@

Library Stdlib.Logic.ChoiceFacts

-

Definitions

+

Definitions

@@ -116,7 +116,7 @@

Library Stdlib.Logic.ChoiceFacts

-

Constructive choice and description

+

Constructive choice and description

@@ -346,7 +346,7 @@

Library Stdlib.Logic.ChoiceFacts

-

Weakly classical choice and description

+

Weakly classical choice and description

@@ -625,7 +625,7 @@

Library Stdlib.Logic.ChoiceFacts

-

Table of contents

+

Table of contents

@@ -682,7 +682,7 @@

Library Stdlib.Logic.ChoiceFacts

-

AC_rel + AC! = AC_fun

+

AC_rel + AC! = AC_fun

@@ -722,7 +722,7 @@

Library Stdlib.Logic.ChoiceFacts

-

Connection between the guarded, non guarded and omniscient choices

+

Connection between the guarded, non guarded and omniscient choices

@@ -733,7 +733,7 @@

Library Stdlib.Logic.ChoiceFacts

irrelevance)
-

AC_rel + PI -> GAC_rel and AC_rel + IGP -> GAC_rel and GAC_rel = OAC_rel

+

AC_rel + PI -> GAC_rel and AC_rel + IGP -> GAC_rel and GAC_rel = OAC_rel

@@ -771,7 +771,7 @@

Library Stdlib.Logic.ChoiceFacts

-

AC_fun + IGP = GAC_fun = OAC_fun = AC_fun + Drinker

+

AC_fun + IGP = GAC_fun = OAC_fun = AC_fun + Drinker

@@ -846,7 +846,7 @@

Library Stdlib.Logic.ChoiceFacts

-

D_iota -> ID_iota and D_epsilon <-> ID_epsilon + Drinker

+

D_iota -> ID_iota and D_epsilon <-> ID_epsilon + Drinker

@@ -890,7 +890,7 @@

Library Stdlib.Logic.ChoiceFacts

-

Derivability of choice for decidable relations with well-ordered codomain

+

Derivability of choice for decidable relations with well-ordered codomain

@@ -923,11 +923,11 @@

Library Stdlib.Logic.ChoiceFacts

-

AC_fun = AC_fun_dep = AC_trunc

+

AC_fun = AC_fun_dep = AC_trunc

-

Choice on dependent and non dependent function types are equivalent

+

Choice on dependent and non dependent function types are equivalent

@@ -966,7 +966,7 @@

Library Stdlib.Logic.ChoiceFacts

-

Functional choice and truncation choice are equivalent

+

Functional choice and truncation choice are equivalent

@@ -983,7 +983,7 @@

Library Stdlib.Logic.ChoiceFacts

-

Reification of dependent and non dependent functional relation are equivalent

+

Reification of dependent and non dependent functional relation are equivalent

@@ -1018,11 +1018,11 @@

Library Stdlib.Logic.ChoiceFacts

-

Non contradiction of constructive descriptions wrt functional axioms of choice

+

Non contradiction of constructive descriptions wrt functional axioms of choice

-

Non contradiction of indefinite description

+

Non contradiction of indefinite description

@@ -1040,7 +1040,7 @@

Library Stdlib.Logic.ChoiceFacts

-

Non contradiction of definite description

+

Non contradiction of definite description

@@ -1084,7 +1084,7 @@

Library Stdlib.Logic.ChoiceFacts

-

Excluded-middle + definite description => computational excluded-middle

+

Excluded-middle + definite description => computational excluded-middle

@@ -1128,7 +1128,7 @@

Library Stdlib.Logic.ChoiceFacts

-

Choice => Dependent choice => Countable choice

+

Choice => Dependent choice => Countable choice

@@ -1148,7 +1148,7 @@

Library Stdlib.Logic.ChoiceFacts

-

About the axiom of choice over setoids

+

About the axiom of choice over setoids

@@ -1160,7 +1160,7 @@

Library Stdlib.Logic.ChoiceFacts

-

Consequences of the choice of a representative in an equivalence class

+

Consequences of the choice of a representative in an equivalence class

@@ -1181,7 +1181,7 @@

Library Stdlib.Logic.ChoiceFacts

-

This is a variant of Diaconescu and Goodman-Myhill theorems

+

This is a variant of Diaconescu and Goodman-Myhill theorems

@@ -1198,7 +1198,7 @@

Library Stdlib.Logic.ChoiceFacts

-

AC_fun_setoid = AC_fun_setoid_gen = AC_fun_setoid_simple

+

AC_fun_setoid = AC_fun_setoid_gen = AC_fun_setoid_simple

@@ -1231,7 +1231,7 @@

Library Stdlib.Logic.ChoiceFacts

-

AC_fun_setoid = AC! + AC_fun_repr

+

AC_fun_setoid = AC! + AC_fun_repr

@@ -1267,7 +1267,7 @@

Library Stdlib.Logic.ChoiceFacts

functional forms, SetoidFunctionalChoice seems strictly stronger
-

AC_fun_setoid = AC_fun + Ext_fun_repr + EM

+

AC_fun_setoid = AC_fun + Ext_fun_repr + EM

@@ -1279,7 +1279,7 @@

Library Stdlib.Logic.ChoiceFacts

-

This is the main theorem in [Carlström04]

+

This is the main theorem in [Carlström04]

@@ -1303,7 +1303,7 @@

Library Stdlib.Logic.ChoiceFacts

-

AC_fun_setoid = AC_fun + Ext_pred_repr + PI

+

AC_fun_setoid = AC_fun + Ext_pred_repr + PI

@@ -1327,7 +1327,7 @@

Library Stdlib.Logic.ChoiceFacts

-

Compatibility notations

+

Compatibility notations

diff --git a/master/stdlib/Stdlib.Logic.ClassicalEpsilon.html b/master/stdlib/Stdlib.Logic.ClassicalEpsilon.html index 07c07057cf..6915086054 100644 --- a/master/stdlib/Stdlib.Logic.ClassicalEpsilon.html +++ b/master/stdlib/Stdlib.Logic.ClassicalEpsilon.html @@ -133,7 +133,7 @@

Library Stdlib.Logic.ClassicalEpsilon

-

Weaker lemmas (compatibility lemmas)

+

Weaker lemmas (compatibility lemmas)

diff --git a/master/stdlib/Stdlib.Logic.ClassicalFacts.html b/master/stdlib/Stdlib.Logic.ClassicalFacts.html index 9fff25e0c5..353b1ba5e6 100644 --- a/master/stdlib/Stdlib.Logic.ClassicalFacts.html +++ b/master/stdlib/Stdlib.Logic.ClassicalFacts.html @@ -118,7 +118,7 @@

Library Stdlib.Logic.ClassicalFacts

-

Prop degeneracy = excluded-middle + prop extensionality

+

Prop degeneracy = excluded-middle + prop extensionality

@@ -194,11 +194,11 @@

Library Stdlib.Logic.ClassicalFacts

-

Classical logic and proof-irrelevance

+

Classical logic and proof-irrelevance

-

CC |- prop ext + A inhabited -> (A = A->A) -> A has fixpoint

+

CC |- prop ext + A inhabited -> (A = A->A) -> A has fixpoint

@@ -251,7 +251,7 @@

Library Stdlib.Logic.ClassicalFacts

-

CC |- prop_ext /\ dep elim on bool -> proof-irrelevance

+

CC |- prop_ext /\ dep elim on bool -> proof-irrelevance

@@ -348,7 +348,7 @@

Library Stdlib.Logic.ClassicalFacts

-

CIC |- prop. ext. -> proof-irrelevance

+

CIC |- prop. ext. -> proof-irrelevance

@@ -402,7 +402,7 @@

Library Stdlib.Logic.ClassicalFacts

-

CC |- excluded-middle + dep elim on bool -> proof-irrelevance

+

CC |- excluded-middle + dep elim on bool -> proof-irrelevance

@@ -574,7 +574,7 @@

Library Stdlib.Logic.ClassicalFacts

-

CIC |- excluded-middle -> proof-irrelevance

+

CIC |- excluded-middle -> proof-irrelevance

@@ -639,7 +639,7 @@

Library Stdlib.Logic.ClassicalFacts

-

Weak classical axioms

+

Weak classical axioms

@@ -661,7 +661,7 @@

Library Stdlib.Logic.ClassicalFacts

-

Weak excluded-middle

+

Weak excluded-middle

@@ -716,7 +716,7 @@

Library Stdlib.Logic.ClassicalFacts

-

Gödel-Dummett axiom

+

Gödel-Dummett axiom

@@ -787,7 +787,7 @@

Library Stdlib.Logic.ClassicalFacts

-

Independence of general premises and drinker's paradox

+

Independence of general premises and drinker's paradox

@@ -963,11 +963,11 @@

Library Stdlib.Logic.ClassicalFacts

-

Axioms equivalent to classical logic

+

Axioms equivalent to classical logic

-

Principle of unrestricted minimization

+

Principle of unrestricted minimization

@@ -1040,7 +1040,7 @@

Library Stdlib.Logic.ClassicalFacts

-

Choice of representatives in a partition of bool

+

Choice of representatives in a partition of bool

diff --git a/master/stdlib/Stdlib.Logic.Diaconescu.html b/master/stdlib/Stdlib.Logic.Diaconescu.html index 3d337e8da2..d18072b507 100644 --- a/master/stdlib/Stdlib.Logic.Diaconescu.html +++ b/master/stdlib/Stdlib.Logic.Diaconescu.html @@ -108,7 +108,7 @@

Library Stdlib.Logic.Diaconescu

-

Pred. Ext. + Rel. Axiom of Choice -> Excluded-Middle

+

Pred. Ext. + Rel. Axiom of Choice -> Excluded-Middle

@@ -204,7 +204,7 @@

Library Stdlib.Logic.Diaconescu

-

Proof-Irrel. + Rel. Axiom of Choice -> Excl.-Middle for Equality

+

Proof-Irrel. + Rel. Axiom of Choice -> Excl.-Middle for Equality

@@ -311,7 +311,7 @@

Library Stdlib.Logic.Diaconescu

-

Extensional Hilbert's epsilon description operator -> Excluded-Middle

+

Extensional Hilbert's epsilon description operator -> Excluded-Middle

diff --git a/master/stdlib/Stdlib.Logic.EqdepFacts.html b/master/stdlib/Stdlib.Logic.EqdepFacts.html index 15b3859e42..c0a085cc48 100644 --- a/master/stdlib/Stdlib.Logic.EqdepFacts.html +++ b/master/stdlib/Stdlib.Logic.EqdepFacts.html @@ -116,7 +116,7 @@

Library Stdlib.Logic.EqdepFacts

-

Definition of dependent equality and equivalence with equality of dependent pairs

+

Definition of dependent equality and equivalence with equality of dependent pairs

@@ -284,7 +284,7 @@

Library Stdlib.Logic.EqdepFacts

-

Eq_rect_eq <-> Eq_dep_eq <-> UIP <-> UIP_refl <-> K

+

Eq_rect_eq <-> Eq_dep_eq <-> UIP <-> UIP_refl <-> K

@@ -510,7 +510,7 @@

Library Stdlib.Logic.EqdepFacts

-

Definition of the functor that builds properties of dependent equalities assuming axiom eq_rect_eq

+

Definition of the functor that builds properties of dependent equalities assuming axiom eq_rect_eq

diff --git a/master/stdlib/Stdlib.Logic.Eqdep_dec.html b/master/stdlib/Stdlib.Logic.Eqdep_dec.html index 4615e7fa19..17db886ef5 100644 --- a/master/stdlib/Stdlib.Logic.Eqdep_dec.html +++ b/master/stdlib/Stdlib.Logic.Eqdep_dec.html @@ -88,7 +88,7 @@

Library Stdlib.Logic.Eqdep_dec

-

Streicher's K and injectivity of dependent pair hold on decidable types

+

Streicher's K and injectivity of dependent pair hold on decidable types

@@ -246,7 +246,7 @@

Library Stdlib.Logic.Eqdep_dec

-

Definition of the functor that builds properties of dependent equalities on decidable sets in Type

+

Definition of the functor that builds properties of dependent equalities on decidable sets in Type

@@ -370,7 +370,7 @@

Library Stdlib.Logic.Eqdep_dec

-

Definition of the functor that builds properties of dependent equalities on decidable sets in Set

+

Definition of the functor that builds properties of dependent equalities on decidable sets in Set

diff --git a/master/stdlib/Stdlib.Logic.ExtensionalityFacts.html b/master/stdlib/Stdlib.Logic.ExtensionalityFacts.html index 2abf9149ca..c666ef7a41 100644 --- a/master/stdlib/Stdlib.Logic.ExtensionalityFacts.html +++ b/master/stdlib/Stdlib.Logic.ExtensionalityFacts.html @@ -105,7 +105,7 @@

Library Stdlib.Logic.ExtensionalityFacts

-

Definitions

+

Definitions

@@ -197,7 +197,7 @@

Library Stdlib.Logic.ExtensionalityFacts

-

Functional extensionality <-> Equality of projections from diagonal

+

Functional extensionality <-> Equality of projections from diagonal

@@ -209,7 +209,7 @@

Library Stdlib.Logic.ExtensionalityFacts

-

Functional extensionality <-> Unicity of bijection inverse

+

Functional extensionality <-> Unicity of bijection inverse

@@ -227,7 +227,7 @@

Library Stdlib.Logic.ExtensionalityFacts

-

Functional extensionality <-> Bijectivity of bijective composition

+

Functional extensionality <-> Bijectivity of bijective composition

diff --git a/master/stdlib/Stdlib.Logic.FinFun.html b/master/stdlib/Stdlib.Logic.FinFun.html index 604634397c..1fee886912 100644 --- a/master/stdlib/Stdlib.Logic.FinFun.html +++ b/master/stdlib/Stdlib.Logic.FinFun.html @@ -49,7 +49,7 @@

Library Stdlib.Logic.FinFun

-

Functions on finite domains

+

Functions on finite domains

diff --git a/master/stdlib/Stdlib.Logic.Hurkens.html b/master/stdlib/Stdlib.Logic.Hurkens.html index 740fc65d6f..b6211eb5ae 100644 --- a/master/stdlib/Stdlib.Logic.Hurkens.html +++ b/master/stdlib/Stdlib.Logic.Hurkens.html @@ -176,7 +176,7 @@

Library Stdlib.Logic.Hurkens

-

A modular proof of Hurkens's paradox.

+

A modular proof of Hurkens's paradox.

@@ -203,7 +203,7 @@

Library Stdlib.Logic.Hurkens

-

Axiomatisation of impredicative universes in a Martin-Löf style

+

Axiomatisation of impredicative universes in a Martin-Löf style

@@ -214,7 +214,7 @@

Library Stdlib.Logic.Hurkens

actual system U-.
-

Large universe

+

Large universe

@@ -223,7 +223,7 @@

Library Stdlib.Logic.Hurkens

-

Closure by small product

+

Closure by small product

@@ -239,7 +239,7 @@

Library Stdlib.Logic.Hurkens

-

Closure by large products

+

Closure by large products

U1 only needs to quantify over itself.
@@ -256,7 +256,7 @@

Library Stdlib.Logic.Hurkens

-

Small universe

+

Small universe

The small universe is an element of the large one.
@@ -266,7 +266,7 @@

Library Stdlib.Logic.Hurkens

-

Closure by small product

+

Closure by small product

U0 does not need reduction rules
@@ -280,7 +280,7 @@

Library Stdlib.Logic.Hurkens

-

Closure by large products

+

Closure by large products

@@ -295,7 +295,7 @@

Library Stdlib.Logic.Hurkens

-

Automating the rewrite rules of our encoding.

+

Automating the rewrite rules of our encoding.

@@ -313,7 +313,7 @@

Library Stdlib.Logic.Hurkens

-

Hurkens's paradox.

+

Hurkens's paradox.

@@ -326,7 +326,7 @@

Library Stdlib.Logic.Hurkens

-

Preliminary definitions

+

Preliminary definitions

@@ -355,7 +355,7 @@

Library Stdlib.Logic.Hurkens

-

Proof

+

Proof

@@ -440,7 +440,7 @@

Library Stdlib.Logic.Hurkens

-

Impredicative universes are not retracts.

+

Impredicative universes are not retracts.

@@ -467,7 +467,7 @@

Library Stdlib.Logic.Hurkens

-

U1 is impredicative

+

U1 is impredicative

@@ -494,7 +494,7 @@

Library Stdlib.Logic.Hurkens

-

U0 is a retract of U1

+

U0 is a retract of U1

@@ -507,7 +507,7 @@

Library Stdlib.Logic.Hurkens

-

Paradox

+

Paradox

@@ -571,7 +571,7 @@

Library Stdlib.Logic.Hurkens

-

Modal fragments of Prop are not retracts

+

Modal fragments of Prop are not retracts

@@ -590,7 +590,7 @@

Library Stdlib.Logic.Hurkens

-

Monadic modality

+

Monadic modality

@@ -613,7 +613,7 @@

Library Stdlib.Logic.Hurkens

-

The universe of modal propositions

+

The universe of modal propositions

@@ -643,7 +643,7 @@

Library Stdlib.Logic.Hurkens

-

Retract of the modal fragment of Prop in a small type

+

Retract of the modal fragment of Prop in a small type

@@ -663,7 +663,7 @@

Library Stdlib.Logic.Hurkens

-

Paradox

+

Paradox

@@ -722,7 +722,7 @@

Library Stdlib.Logic.Hurkens

-

The negative fragment of Prop is not a retract

+

The negative fragment of Prop is not a retract

@@ -739,7 +739,7 @@

Library Stdlib.Logic.Hurkens

-

The universe of negative propositions.

+

The universe of negative propositions.

@@ -755,7 +755,7 @@

Library Stdlib.Logic.Hurkens

-

Retract of the negative fragment of Prop in a small type

+

Retract of the negative fragment of Prop in a small type

@@ -775,7 +775,7 @@

Library Stdlib.Logic.Hurkens

-

Paradox

+

Paradox

@@ -806,7 +806,7 @@

Library Stdlib.Logic.Hurkens

-

Prop is not a retract

+

Prop is not a retract

@@ -823,7 +823,7 @@

Library Stdlib.Logic.Hurkens

-

The universe of propositions.

+

The universe of propositions.

@@ -839,7 +839,7 @@

Library Stdlib.Logic.Hurkens

-

Retract of Prop in a small type, using the identity modality.

+

Retract of Prop in a small type, using the identity modality.

@@ -855,7 +855,7 @@

Library Stdlib.Logic.Hurkens

-

Paradox

+

Paradox

@@ -886,7 +886,7 @@

Library Stdlib.Logic.Hurkens

-

Retract of Prop in a small type

+

Retract of Prop in a small type

@@ -904,7 +904,7 @@

Library Stdlib.Logic.Hurkens

-

Paradox

+

Paradox

@@ -931,7 +931,7 @@

Library Stdlib.Logic.Hurkens

-

Large universes are not retracts of Prop.

+

Large universes are not retracts of Prop.

@@ -956,7 +956,7 @@

Library Stdlib.Logic.Hurkens

-

Assumption of a retract from Type into Prop

+

Assumption of a retract from Type into Prop

@@ -970,7 +970,7 @@

Library Stdlib.Logic.Hurkens

-

Paradox

+

Paradox

@@ -1025,7 +1025,7 @@

Library Stdlib.Logic.Hurkens

-

A<>Type

+

A<>Type

@@ -1046,7 +1046,7 @@

Library Stdlib.Logic.Hurkens

-

Universe U is equal to one of its elements.

+

Universe U is equal to one of its elements.

@@ -1060,7 +1060,7 @@

Library Stdlib.Logic.Hurkens

-

Universe U is a retract of A

+

Universe U is a retract of A

@@ -1150,7 +1150,7 @@

Library Stdlib.Logic.Hurkens

-

Prop<>Type.

+

Prop<>Type.

diff --git a/master/stdlib/Stdlib.Logic.PropExtensionalityFacts.html b/master/stdlib/Stdlib.Logic.PropExtensionalityFacts.html index 4a07e71235..65d5520aaa 100644 --- a/master/stdlib/Stdlib.Logic.PropExtensionalityFacts.html +++ b/master/stdlib/Stdlib.Logic.PropExtensionalityFacts.html @@ -117,7 +117,7 @@

Library Stdlib.Logic.PropExtensionalityFacts

-

Definitions

+

Definitions

@@ -181,11 +181,11 @@

Library Stdlib.Logic.PropExtensionalityFacts

-

Propositional and predicate extensionality

+

Propositional and predicate extensionality

-

Predicate extensionality <-> Propositional extensionality + Propositional functional extensionality

+

Predicate extensionality <-> Propositional extensionality + Propositional functional extensionality

@@ -208,7 +208,7 @@

Library Stdlib.Logic.PropExtensionalityFacts

-

Propositional extensionality and provable proposition extensionality

+

Propositional extensionality and provable proposition extensionality

@@ -220,7 +220,7 @@

Library Stdlib.Logic.PropExtensionalityFacts

-

Propositional extensionality and refutable proposition extensionality

+

Propositional extensionality and refutable proposition extensionality

diff --git a/master/stdlib/Stdlib.Logic.PropFacts.html b/master/stdlib/Stdlib.Logic.PropFacts.html index 0487abc939..c79f765906 100644 --- a/master/stdlib/Stdlib.Logic.PropFacts.html +++ b/master/stdlib/Stdlib.Logic.PropFacts.html @@ -49,7 +49,7 @@

Library Stdlib.Logic.PropFacts

-

Basic facts about Prop as a type

+

Basic facts about Prop as a type

diff --git a/master/stdlib/Stdlib.Logic.SetIsType.html b/master/stdlib/Stdlib.Logic.SetIsType.html index 3c521cdc2a..c6f99d6462 100644 --- a/master/stdlib/Stdlib.Logic.SetIsType.html +++ b/master/stdlib/Stdlib.Logic.SetIsType.html @@ -49,7 +49,7 @@

Library Stdlib.Logic.SetIsType

-

The Set universe seen as a synonym for Type

+

The Set universe seen as a synonym for Type

diff --git a/master/stdlib/Stdlib.MSets.MSetAVL.html b/master/stdlib/Stdlib.MSets.MSetAVL.html index 0c60aff02c..e3a50aea70 100644 --- a/master/stdlib/Stdlib.MSets.MSetAVL.html +++ b/master/stdlib/Stdlib.MSets.MSetAVL.html @@ -49,7 +49,7 @@

Library Stdlib.MSets.MSetAVL

-

MSetAVL : Implementation of MSetInterface via AVL trees

+

MSetAVL : Implementation of MSetInterface via AVL trees

@@ -91,7 +91,7 @@

Library Stdlib.MSets.MSetAVL

-

Ops : the pure functions

+

Ops : the pure functions

@@ -105,7 +105,7 @@

Library Stdlib.MSets.MSetAVL

-

Generic trees instantiated with integer height

+

Generic trees instantiated with integer height

@@ -125,7 +125,7 @@

Library Stdlib.MSets.MSetAVL

-

Height of trees

+

Height of trees

@@ -141,7 +141,7 @@

Library Stdlib.MSets.MSetAVL

-

Singleton set

+

Singleton set

@@ -153,7 +153,7 @@

Library Stdlib.MSets.MSetAVL

-

Helper functions

+

Helper functions

@@ -216,7 +216,7 @@

Library Stdlib.MSets.MSetAVL

-

Insertion

+

Insertion

@@ -236,7 +236,7 @@

Library Stdlib.MSets.MSetAVL

-

Join

+

Join

@@ -265,7 +265,7 @@

Library Stdlib.MSets.MSetAVL

-

Extraction of minimum element

+

Extraction of minimum element

@@ -289,7 +289,7 @@

Library Stdlib.MSets.MSetAVL

-

Merging two trees

+

Merging two trees

@@ -313,7 +313,7 @@

Library Stdlib.MSets.MSetAVL

-

Deletion

+

Deletion

@@ -333,7 +333,7 @@

Library Stdlib.MSets.MSetAVL

-

Concatenation

+

Concatenation

@@ -357,7 +357,7 @@

Library Stdlib.MSets.MSetAVL

-

Splitting

+

Splitting

@@ -397,7 +397,7 @@

Library Stdlib.MSets.MSetAVL

-

Intersection

+

Intersection

@@ -416,7 +416,7 @@

Library Stdlib.MSets.MSetAVL

-

Difference

+

Difference

@@ -435,7 +435,7 @@

Library Stdlib.MSets.MSetAVL

-

Union

+

Union

@@ -466,7 +466,7 @@

Library Stdlib.MSets.MSetAVL

-

Filter

+

Filter

@@ -484,7 +484,7 @@

Library Stdlib.MSets.MSetAVL

-

Partition

+

Partition

@@ -507,7 +507,7 @@

Library Stdlib.MSets.MSetAVL

-

MakeRaw

+

MakeRaw

@@ -780,7 +780,7 @@

Library Stdlib.MSets.MSetAVL

-

Singleton set

+

Singleton set

@@ -796,7 +796,7 @@

Library Stdlib.MSets.MSetAVL

-

Helper functions

+

Helper functions

@@ -823,7 +823,7 @@

Library Stdlib.MSets.MSetAVL

-

Insertion

+

Insertion

@@ -847,7 +847,7 @@

Library Stdlib.MSets.MSetAVL

-

Join

+

Join

@@ -886,7 +886,7 @@

Library Stdlib.MSets.MSetAVL

-

Extraction of minimum element

+

Extraction of minimum element

@@ -910,7 +910,7 @@

Library Stdlib.MSets.MSetAVL

-

Merging two trees

+

Merging two trees

@@ -929,7 +929,7 @@

Library Stdlib.MSets.MSetAVL

-

Deletion

+

Deletion

@@ -946,7 +946,7 @@

Library Stdlib.MSets.MSetAVL

-

Concatenation

+

Concatenation

@@ -965,7 +965,7 @@

Library Stdlib.MSets.MSetAVL

-

Splitting

+

Splitting

@@ -997,7 +997,7 @@

Library Stdlib.MSets.MSetAVL

-

Intersection

+

Intersection

@@ -1027,7 +1027,7 @@

Library Stdlib.MSets.MSetAVL

-

Difference

+

Difference

@@ -1048,7 +1048,7 @@

Library Stdlib.MSets.MSetAVL

-

Union

+

Union

@@ -1065,7 +1065,7 @@

Library Stdlib.MSets.MSetAVL

-

Filter

+

Filter

@@ -1087,7 +1087,7 @@

Library Stdlib.MSets.MSetAVL

-

Partition

+

Partition

@@ -1124,7 +1124,7 @@

Library Stdlib.MSets.MSetAVL

-

Encapsulation

+

Encapsulation

diff --git a/master/stdlib/Stdlib.MSets.MSetDecide.html b/master/stdlib/Stdlib.MSets.MSetDecide.html index 031de937dc..5e2d30cb76 100644 --- a/master/stdlib/Stdlib.MSets.MSetDecide.html +++ b/master/stdlib/Stdlib.MSets.MSetDecide.html @@ -75,7 +75,7 @@

Library Stdlib.MSets.MSetDecide

-

Overview

+

Overview

This functor defines the tactic fsetdec, which will solve any valid goal of the form @@ -181,7 +181,7 @@

Library Stdlib.MSets.MSetDecide

-

Facts and Tactics for Propositional Logic

+

Facts and Tactics for Propositional Logic

These lemmas and tactics are in a module so that they do not affect the namespace if you import the enclosing @@ -196,18 +196,18 @@

Library Stdlib.MSets.MSetDecide

-

Lemmas and Tactics About Decidable Propositions

+

Lemmas and Tactics About Decidable Propositions

-

Propositional Equivalences Involving Negation

+

Propositional Equivalences Involving Negation

These are all written with the unfolded form of negation, since I am not sure if setoid rewriting will always perform conversion.
-

Tactics for Negations

+

Tactics for Negations

@@ -458,7 +458,7 @@

Library Stdlib.MSets.MSetDecide

-

Auxiliary Tactics

+

Auxiliary Tactics

Again, these lemmas and tactics are in a module so that they do not affect the namespace if you import the @@ -471,7 +471,7 @@

Library Stdlib.MSets.MSetDecide

-

Generic Tactics

+

Generic Tactics

We begin by defining a few generic, useful tactics.
@@ -588,7 +588,7 @@

Library Stdlib.MSets.MSetDecide

-

Discarding Irrelevant Hypotheses

+

Discarding Irrelevant Hypotheses

We will want to clear the context of any non-MSet-related hypotheses in order to increase the @@ -668,7 +668,7 @@

Library Stdlib.MSets.MSetDecide

-

Turning Set Operators into Propositional Connectives

+

Turning Set Operators into Propositional Connectives

The lemmas from MSetFacts will be used to break down set operations into propositional formulas built over @@ -694,7 +694,7 @@

Library Stdlib.MSets.MSetDecide

-

Decidability of MSet Propositions

+

Decidability of MSet Propositions

@@ -729,7 +729,7 @@

Library Stdlib.MSets.MSetDecide

-

Normalizing Propositions About Equality

+

Normalizing Propositions About Equality

We have to deal with the fact that E.eq may be convertible with Coq's equality. Thus, we will find the @@ -812,7 +812,7 @@

Library Stdlib.MSets.MSetDecide

-

Considering Decidability of Base Propositions

+

Considering Decidability of Base Propositions

This tactic adds assertions about the decidability of E.eq and In to the context. This is necessary for @@ -861,7 +861,7 @@

Library Stdlib.MSets.MSetDecide

-

Handling Empty, Subset, and Equal

+

Handling Empty, Subset, and Equal

This tactic instantiates universally quantified hypotheses (which arise from the unfolding of Empty, @@ -909,7 +909,7 @@

Library Stdlib.MSets.MSetDecide

-

The Core fsetdec Auxiliary Tactics

+

The Core fsetdec Auxiliary Tactics

@@ -951,7 +951,7 @@

Library Stdlib.MSets.MSetDecide

-

The fsetdec Tactic

+

The fsetdec Tactic

Here is the top-level tactic (the only one intended for clients of this library). It's specification is given at @@ -1065,7 +1065,7 @@

Library Stdlib.MSets.MSetDecide

-

Examples

+

Examples

diff --git a/master/stdlib/Stdlib.MSets.MSetEqProperties.html b/master/stdlib/Stdlib.MSets.MSetEqProperties.html index 067a8890b7..88296c183d 100644 --- a/master/stdlib/Stdlib.MSets.MSetEqProperties.html +++ b/master/stdlib/Stdlib.MSets.MSetEqProperties.html @@ -49,7 +49,7 @@

Library Stdlib.MSets.MSetEqProperties

-

Finite sets library

+

Finite sets library

diff --git a/master/stdlib/Stdlib.MSets.MSetFacts.html b/master/stdlib/Stdlib.MSets.MSetFacts.html index 653d308cb8..49d132e28a 100644 --- a/master/stdlib/Stdlib.MSets.MSetFacts.html +++ b/master/stdlib/Stdlib.MSets.MSetFacts.html @@ -49,7 +49,7 @@

Library Stdlib.MSets.MSetFacts

-

Finite sets library

+

Finite sets library

@@ -88,7 +88,7 @@

Library Stdlib.MSets.MSetFacts

-

Specifications written using implications :

+

Specifications written using implications :

this used to be the default interface.
@@ -205,7 +205,7 @@

Library Stdlib.MSets.MSetFacts

-

Specifications written using equivalences :

+

Specifications written using equivalences :

this is now provided by the default interface.
@@ -294,7 +294,7 @@

Library Stdlib.MSets.MSetFacts

-

Specifications written using boolean predicates

+

Specifications written using boolean predicates

@@ -358,7 +358,7 @@

Library Stdlib.MSets.MSetFacts

-

Declarations of morphisms with respects to E.eq and Equal

+

Declarations of morphisms with respects to E.eq and Equal

diff --git a/master/stdlib/Stdlib.MSets.MSetGenTree.html b/master/stdlib/Stdlib.MSets.MSetGenTree.html index a795b9e3d2..c1053bd4ed 100644 --- a/master/stdlib/Stdlib.MSets.MSetGenTree.html +++ b/master/stdlib/Stdlib.MSets.MSetGenTree.html @@ -49,7 +49,7 @@

Library Stdlib.MSets.MSetGenTree

-

MSetGenTree : sets via generic trees

+

MSetGenTree : sets via generic trees

@@ -107,7 +107,7 @@

Library Stdlib.MSets.MSetGenTree

-

Ops : the pure functions

+

Ops : the pure functions

@@ -129,7 +129,7 @@

Library Stdlib.MSets.MSetGenTree

-

The empty set and emptyness test

+

The empty set and emptyness test

@@ -148,7 +148,7 @@

Library Stdlib.MSets.MSetGenTree

-

Membership test

+

Membership test

@@ -173,7 +173,7 @@

Library Stdlib.MSets.MSetGenTree

-

Minimal, maximal, arbitrary elements

+

Minimal, maximal, arbitrary elements

@@ -201,7 +201,7 @@

Library Stdlib.MSets.MSetGenTree

-

Iteration on elements

+

Iteration on elements

@@ -258,7 +258,7 @@

Library Stdlib.MSets.MSetGenTree

-

Testing universal or existential properties.

+

Testing universal or existential properties.

@@ -283,7 +283,7 @@

Library Stdlib.MSets.MSetGenTree

-

Comparison of trees

+

Comparison of trees

@@ -390,7 +390,7 @@

Library Stdlib.MSets.MSetGenTree

-

Subset test

+

Subset test

@@ -449,7 +449,7 @@

Library Stdlib.MSets.MSetGenTree

-

Props : correctness proofs of these generic operations

+

Props : correctness proofs of these generic operations

@@ -461,7 +461,7 @@

Library Stdlib.MSets.MSetGenTree

-

Occurrence in a tree

+

Occurrence in a tree

@@ -479,7 +479,7 @@

Library Stdlib.MSets.MSetGenTree

-

Some shortcuts

+

Some shortcuts

@@ -495,7 +495,7 @@

Library Stdlib.MSets.MSetGenTree

-

Binary search trees

+

Binary search trees

@@ -573,7 +573,7 @@

Library Stdlib.MSets.MSetGenTree

-

Known facts about ordered types

+

Known facts about ordered types

@@ -585,7 +585,7 @@

Library Stdlib.MSets.MSetGenTree

-

Automation and dedicated tactics

+

Automation and dedicated tactics

@@ -692,7 +692,7 @@

Library Stdlib.MSets.MSetGenTree

-

Basic results about In

+

Basic results about In

@@ -790,7 +790,7 @@

Library Stdlib.MSets.MSetGenTree

-

Empty set

+

Empty set

@@ -806,7 +806,7 @@

Library Stdlib.MSets.MSetGenTree

-

Emptyness test

+

Emptyness test

@@ -818,7 +818,7 @@

Library Stdlib.MSets.MSetGenTree

-

Membership

+

Membership

@@ -830,7 +830,7 @@

Library Stdlib.MSets.MSetGenTree

-

Minimal and maximal elements

+

Minimal and maximal elements

@@ -870,7 +870,7 @@

Library Stdlib.MSets.MSetGenTree

-

Elements

+

Elements

@@ -946,7 +946,7 @@

Library Stdlib.MSets.MSetGenTree

-

for_all and exists

+

for_all and exists

@@ -963,7 +963,7 @@

Library Stdlib.MSets.MSetGenTree

-

Fold

+

Fold

@@ -980,7 +980,7 @@

Library Stdlib.MSets.MSetGenTree

-

Subset

+

Subset

@@ -1005,7 +1005,7 @@

Library Stdlib.MSets.MSetGenTree

-

Comparison

+

Comparison

@@ -1107,7 +1107,7 @@

Library Stdlib.MSets.MSetGenTree

-

Equality test

+

Equality test

@@ -1120,7 +1120,7 @@

Library Stdlib.MSets.MSetGenTree

-

A few results about mindepth and maxdepth

+

A few results about mindepth and maxdepth

diff --git a/master/stdlib/Stdlib.MSets.MSetInterface.html b/master/stdlib/Stdlib.MSets.MSetInterface.html index a5d9417b5d..e33ce07b90 100644 --- a/master/stdlib/Stdlib.MSets.MSetInterface.html +++ b/master/stdlib/Stdlib.MSets.MSetInterface.html @@ -49,7 +49,7 @@

Library Stdlib.MSets.MSetInterface

-

Finite set library

+

Finite set library

@@ -318,7 +318,7 @@

Library Stdlib.MSets.MSetInterface

-

Functorial signature for weak sets

+

Functorial signature for weak sets

@@ -432,7 +432,7 @@

Library Stdlib.MSets.MSetInterface

-

Static signature for weak sets

+

Static signature for weak sets

@@ -452,7 +452,7 @@

Library Stdlib.MSets.MSetInterface

-

Functorial signature for sets on ordered elements

+

Functorial signature for sets on ordered elements

@@ -564,7 +564,7 @@

Library Stdlib.MSets.MSetInterface

-

Static signature for sets on ordered elements

+

Static signature for sets on ordered elements

@@ -587,7 +587,7 @@

Library Stdlib.MSets.MSetInterface

-

Some subtyping tests

+

Some subtyping tests

 WSetsOn ---> WSets
@@ -604,7 +604,7 @@ 

Library Stdlib.MSets.MSetInterface

-

Signatures for set representations with ill-formed values.

+

Signatures for set representations with ill-formed values.

diff --git a/master/stdlib/Stdlib.MSets.MSetList.html b/master/stdlib/Stdlib.MSets.MSetList.html index 019bdd227a..1f7b9d6159 100644 --- a/master/stdlib/Stdlib.MSets.MSetList.html +++ b/master/stdlib/Stdlib.MSets.MSetList.html @@ -49,7 +49,7 @@

Library Stdlib.MSets.MSetList

-

Finite sets library

+

Finite sets library

@@ -66,7 +66,7 @@

Library Stdlib.MSets.MSetList

-

Functions over lists

+

Functions over lists

@@ -94,7 +94,7 @@

Library Stdlib.MSets.MSetList

-

The set operations.

+

The set operations.

@@ -302,7 +302,7 @@

Library Stdlib.MSets.MSetList

-

Proofs of set operation specifications.

+

Proofs of set operation specifications.

@@ -643,7 +643,7 @@

Library Stdlib.MSets.MSetList

-

Encapsulation

+

Encapsulation

diff --git a/master/stdlib/Stdlib.MSets.MSetProperties.html b/master/stdlib/Stdlib.MSets.MSetProperties.html index e5d096d748..79a7a99062 100644 --- a/master/stdlib/Stdlib.MSets.MSetProperties.html +++ b/master/stdlib/Stdlib.MSets.MSetProperties.html @@ -49,7 +49,7 @@

Library Stdlib.MSets.MSetProperties

-

Finite sets library

+

Finite sets library

@@ -342,7 +342,7 @@

Library Stdlib.MSets.MSetProperties

-

Properties of elements

+

Properties of elements

@@ -357,7 +357,7 @@

Library Stdlib.MSets.MSetProperties

-

Conversions between lists and sets

+

Conversions between lists and sets

@@ -381,7 +381,7 @@

Library Stdlib.MSets.MSetProperties

-

Fold

+

Fold

@@ -409,7 +409,7 @@

Library Stdlib.MSets.MSetProperties

-

Induction principles for fold (contributed by S. Lescuyer)

+

Induction principles for fold (contributed by S. Lescuyer)

@@ -515,7 +515,7 @@

Library Stdlib.MSets.MSetProperties

-

Alternative (weaker) specifications for fold

+

Alternative (weaker) specifications for fold

@@ -587,7 +587,7 @@

Library Stdlib.MSets.MSetProperties

-

Fold is a morphism

+

Fold is a morphism

@@ -604,7 +604,7 @@

Library Stdlib.MSets.MSetProperties

-

Fold and other set operators

+

Fold and other set operators

@@ -656,11 +656,11 @@

Library Stdlib.MSets.MSetProperties

-

Cardinal

+

Cardinal

-

Characterization of cardinal in terms of fold

+

Characterization of cardinal in terms of fold

@@ -672,7 +672,7 @@

Library Stdlib.MSets.MSetProperties

-

Old specifications for cardinal.

+

Old specifications for cardinal.

@@ -695,7 +695,7 @@

Library Stdlib.MSets.MSetProperties

-

Cardinal and (non-)emptiness

+

Cardinal and (non-)emptiness

@@ -720,7 +720,7 @@

Library Stdlib.MSets.MSetProperties

-

Cardinal is a morphism

+

Cardinal is a morphism

@@ -740,7 +740,7 @@

Library Stdlib.MSets.MSetProperties

-

Cardinal and set operators

+

Cardinal and set operators

diff --git a/master/stdlib/Stdlib.MSets.MSetRBT.html b/master/stdlib/Stdlib.MSets.MSetRBT.html index 6815cd56ba..4173cb9942 100644 --- a/master/stdlib/Stdlib.MSets.MSetRBT.html +++ b/master/stdlib/Stdlib.MSets.MSetRBT.html @@ -49,7 +49,7 @@

Library Stdlib.MSets.MSetRBT

-

MSetRBT : Implementation of MSetInterface via Red-Black trees

+

MSetRBT : Implementation of MSetInterface via Red-Black trees

@@ -153,7 +153,7 @@

Library Stdlib.MSets.MSetRBT

-

Ops : the pure functions

+

Ops : the pure functions

@@ -165,7 +165,7 @@

Library Stdlib.MSets.MSetRBT

-

Generic trees instantiated with color

+

Generic trees instantiated with color

@@ -187,7 +187,7 @@

Library Stdlib.MSets.MSetRBT

-

Basic tree

+

Basic tree

@@ -199,7 +199,7 @@

Library Stdlib.MSets.MSetRBT

-

Changing root color

+

Changing root color

@@ -222,7 +222,7 @@

Library Stdlib.MSets.MSetRBT

-

Balancing

+

Balancing

@@ -303,7 +303,7 @@

Library Stdlib.MSets.MSetRBT

-

Insertion

+

Insertion

@@ -335,7 +335,7 @@

Library Stdlib.MSets.MSetRBT

-

Deletion

+

Deletion

@@ -395,7 +395,7 @@

Library Stdlib.MSets.MSetRBT

-

Removing minimal element

+

Removing minimal element

@@ -425,7 +425,7 @@

Library Stdlib.MSets.MSetRBT

-

Tree-ification

+

Tree-ification

@@ -488,7 +488,7 @@

Library Stdlib.MSets.MSetRBT

-

Filtering

+

Filtering

@@ -526,7 +526,7 @@

Library Stdlib.MSets.MSetRBT

-

Union, intersection, difference

+

Union, intersection, difference

@@ -686,7 +686,7 @@

Library Stdlib.MSets.MSetRBT

-

MakeRaw : the pure functions and their specifications

+

MakeRaw : the pure functions and their specifications

@@ -724,7 +724,7 @@

Library Stdlib.MSets.MSetRBT

-

Singleton set

+

Singleton set

@@ -740,7 +740,7 @@

Library Stdlib.MSets.MSetRBT

-

makeBlack, MakeRed

+

makeBlack, MakeRed

@@ -763,7 +763,7 @@

Library Stdlib.MSets.MSetRBT

-

Generic handling for red-matching and red-red-matching

+

Generic handling for red-matching and red-red-matching

@@ -888,7 +888,7 @@

Library Stdlib.MSets.MSetRBT

-

Balancing for insertion

+

Balancing for insertion

@@ -934,7 +934,7 @@

Library Stdlib.MSets.MSetRBT

-

Insertion

+

Insertion

@@ -967,7 +967,7 @@

Library Stdlib.MSets.MSetRBT

-

Balancing for deletion

+

Balancing for deletion

@@ -997,7 +997,7 @@

Library Stdlib.MSets.MSetRBT

-

Append for deletion

+

Append for deletion

@@ -1050,7 +1050,7 @@

Library Stdlib.MSets.MSetRBT

-

Deletion

+

Deletion

@@ -1081,7 +1081,7 @@

Library Stdlib.MSets.MSetRBT

-

Removing the minimal element

+

Removing the minimal element

@@ -1110,7 +1110,7 @@

Library Stdlib.MSets.MSetRBT

-

Treeify

+

Treeify

@@ -1162,7 +1162,7 @@

Library Stdlib.MSets.MSetRBT

-

Filter

+

Filter

@@ -1188,7 +1188,7 @@

Library Stdlib.MSets.MSetRBT

-

Partition

+

Partition

@@ -1224,7 +1224,7 @@

Library Stdlib.MSets.MSetRBT

-

An invariant for binary list functions with accumulator.

+

An invariant for binary list functions with accumulator.

@@ -1271,7 +1271,7 @@

Library Stdlib.MSets.MSetRBT

-

union

+

union

@@ -1319,7 +1319,7 @@

Library Stdlib.MSets.MSetRBT

-

inter

+

inter

@@ -1360,7 +1360,7 @@

Library Stdlib.MSets.MSetRBT

-

difference

+

difference

@@ -1409,7 +1409,7 @@

Library Stdlib.MSets.MSetRBT

-

Balancing properties

+

Balancing properties

@@ -1432,7 +1432,7 @@

Library Stdlib.MSets.MSetRBT

-

Red-Black invariants

+

Red-Black invariants

@@ -1503,7 +1503,7 @@

Library Stdlib.MSets.MSetRBT

-

Basic tactics and results about red-black

+

Basic tactics and results about red-black

@@ -1538,7 +1538,7 @@

Library Stdlib.MSets.MSetRBT

-

A Red-Black tree has indeed a logarithmic depth

+

A Red-Black tree has indeed a logarithmic depth

@@ -1564,7 +1564,7 @@

Library Stdlib.MSets.MSetRBT

-

Singleton

+

Singleton

@@ -1576,7 +1576,7 @@

Library Stdlib.MSets.MSetRBT

-

makeBlack and makeRed

+

makeBlack and makeRed

@@ -1592,7 +1592,7 @@

Library Stdlib.MSets.MSetRBT

-

Balancing

+

Balancing

@@ -1629,7 +1629,7 @@

Library Stdlib.MSets.MSetRBT

-

Insertion

+

Insertion

@@ -1662,7 +1662,7 @@

Library Stdlib.MSets.MSetRBT

-

Deletion

+

Deletion

@@ -1693,7 +1693,7 @@

Library Stdlib.MSets.MSetRBT

-

Treeify

+

Treeify

@@ -1740,7 +1740,7 @@

Library Stdlib.MSets.MSetRBT

-

Filtering

+

Filtering

@@ -1761,7 +1761,7 @@

Library Stdlib.MSets.MSetRBT

-

Union, intersection, difference

+

Union, intersection, difference

@@ -1790,7 +1790,7 @@

Library Stdlib.MSets.MSetRBT

-

Final Encapsulation

+

Final Encapsulation

diff --git a/master/stdlib/Stdlib.MSets.MSetToFiniteSet.html b/master/stdlib/Stdlib.MSets.MSetToFiniteSet.html index 2e49a84496..0c72e4d3d9 100644 --- a/master/stdlib/Stdlib.MSets.MSetToFiniteSet.html +++ b/master/stdlib/Stdlib.MSets.MSetToFiniteSet.html @@ -49,7 +49,7 @@

Library Stdlib.MSets.MSetToFiniteSet

-

Finite sets library : conversion to old Finite_sets

+

Finite sets library : conversion to old Finite_sets

@@ -62,7 +62,7 @@

Library Stdlib.MSets.MSetToFiniteSet

-

Going from MSets with usual Leibniz equality

+

Going from MSets with usual Leibniz equality

to the good old Ensembles and Finite_sets theory.
diff --git a/master/stdlib/Stdlib.MSets.MSetWeakList.html b/master/stdlib/Stdlib.MSets.MSetWeakList.html index 9b4dd28ce1..d5f131b161 100644 --- a/master/stdlib/Stdlib.MSets.MSetWeakList.html +++ b/master/stdlib/Stdlib.MSets.MSetWeakList.html @@ -49,7 +49,7 @@

Library Stdlib.MSets.MSetWeakList

-

Finite sets library

+

Finite sets library

@@ -69,7 +69,7 @@

Library Stdlib.MSets.MSetWeakList

-

Functions over lists

+

Functions over lists

@@ -79,7 +79,7 @@

Library Stdlib.MSets.MSetWeakList

And the functions returning sets are proved to preserve this invariant.
-

The set operations.

+

The set operations.

@@ -194,7 +194,7 @@

Library Stdlib.MSets.MSetWeakList

-

Proofs of set operation specifications.

+

Proofs of set operation specifications.

@@ -426,7 +426,7 @@

Library Stdlib.MSets.MSetWeakList

-

Encapsulation

+

Encapsulation

diff --git a/master/stdlib/Stdlib.NArith.BinNat.html b/master/stdlib/Stdlib.NArith.BinNat.html index ff302d530f..3bab6637c4 100644 --- a/master/stdlib/Stdlib.NArith.BinNat.html +++ b/master/stdlib/Stdlib.NArith.BinNat.html @@ -55,7 +55,7 @@

Library Stdlib.NArith.BinNat

-

Binary natural numbers, operations and properties

+

Binary natural numbers, operations and properties

@@ -895,7 +895,7 @@

Library Stdlib.NArith.BinNat

-

Properties of iter

+

Properties of iter

diff --git a/master/stdlib/Stdlib.NArith.BinNatDef.html b/master/stdlib/Stdlib.NArith.BinNatDef.html index d647923b46..ad9c79c018 100644 --- a/master/stdlib/Stdlib.NArith.BinNatDef.html +++ b/master/stdlib/Stdlib.NArith.BinNatDef.html @@ -61,7 +61,7 @@

Library Stdlib.NArith.BinNatDef

-

Binary natural numbers, definitions of operations

+

Binary natural numbers, definitions of operations

@@ -76,7 +76,7 @@

Library Stdlib.NArith.BinNatDef

-

Nicer name N.pos for constructor Npos

+

Nicer name N.pos for constructor Npos

@@ -88,7 +88,7 @@

Library Stdlib.NArith.BinNatDef

-

Constants

+

Constants

@@ -102,7 +102,7 @@

Library Stdlib.NArith.BinNatDef

-

Operation x -> 2*x+1

+

Operation x -> 2*x+1

@@ -118,7 +118,7 @@

Library Stdlib.NArith.BinNatDef

-

Operation x -> 2*x

+

Operation x -> 2*x

@@ -134,7 +134,7 @@

Library Stdlib.NArith.BinNatDef

-

Successor

+

Successor

@@ -150,7 +150,7 @@

Library Stdlib.NArith.BinNatDef

-

Predecessor

+

Predecessor

@@ -166,7 +166,7 @@

Library Stdlib.NArith.BinNatDef

-

The successor of a N can be seen as a positive

+

The successor of a N can be seen as a positive

@@ -182,7 +182,7 @@

Library Stdlib.NArith.BinNatDef

-

Addition

+

Addition

diff --git a/master/stdlib/Stdlib.NArith.Nnat.html b/master/stdlib/Stdlib.NArith.Nnat.html index d042c43122..41306b37b7 100644 --- a/master/stdlib/Stdlib.NArith.Nnat.html +++ b/master/stdlib/Stdlib.NArith.Nnat.html @@ -52,7 +52,7 @@

Library Stdlib.NArith.Nnat

-

Conversions from N to nat

+

Conversions from N to nat

@@ -168,7 +168,7 @@

Library Stdlib.NArith.Nnat

-

Conversions from nat to N

+

Conversions from nat to N

diff --git a/master/stdlib/Stdlib.Numbers.AltBinNotations.html b/master/stdlib/Stdlib.Numbers.AltBinNotations.html index a720e58517..f1cb1ba923 100644 --- a/master/stdlib/Stdlib.Numbers.AltBinNotations.html +++ b/master/stdlib/Stdlib.Numbers.AltBinNotations.html @@ -49,7 +49,7 @@

Library Stdlib.Numbers.AltBinNotations

-

Alternative Binary Number Notations

+

Alternative Binary Number Notations

diff --git a/master/stdlib/Stdlib.Numbers.BinNums.html b/master/stdlib/Stdlib.Numbers.BinNums.html index 5bd2426988..dd16781cbf 100644 --- a/master/stdlib/Stdlib.Numbers.BinNums.html +++ b/master/stdlib/Stdlib.Numbers.BinNums.html @@ -49,7 +49,7 @@

Library Stdlib.Numbers.BinNums

-

Binary Numerical Datatypes

+

Binary Numerical Datatypes

diff --git a/master/stdlib/Stdlib.Numbers.Cyclic.Abstract.CyclicAxioms.html b/master/stdlib/Stdlib.Numbers.Cyclic.Abstract.CyclicAxioms.html index 66b3239a58..eeb1269e85 100644 --- a/master/stdlib/Stdlib.Numbers.Cyclic.Abstract.CyclicAxioms.html +++ b/master/stdlib/Stdlib.Numbers.Cyclic.Abstract.CyclicAxioms.html @@ -49,7 +49,7 @@

Library Stdlib.Numbers.Cyclic.Abstract.CyclicAxioms

-

Signature and specification of bounded integers

+

Signature and specification of bounded integers

diff --git a/master/stdlib/Stdlib.Numbers.Cyclic.Abstract.NZCyclic.html b/master/stdlib/Stdlib.Numbers.Cyclic.Abstract.NZCyclic.html index 2b1c5ae28f..26dd77fadd 100644 --- a/master/stdlib/Stdlib.Numbers.Cyclic.Abstract.NZCyclic.html +++ b/master/stdlib/Stdlib.Numbers.Cyclic.Abstract.NZCyclic.html @@ -57,7 +57,7 @@

Library Stdlib.Numbers.Cyclic.Abstract.NZCyclic

-

From CyclicType to NZAxiomsSig

+

From CyclicType to NZAxiomsSig

diff --git a/master/stdlib/Stdlib.Numbers.Cyclic.Int63.Cyclic63.html b/master/stdlib/Stdlib.Numbers.Cyclic.Int63.Cyclic63.html index be950185a0..fb368ee825 100644 --- a/master/stdlib/Stdlib.Numbers.Cyclic.Int63.Cyclic63.html +++ b/master/stdlib/Stdlib.Numbers.Cyclic.Int63.Cyclic63.html @@ -49,7 +49,7 @@

Library Stdlib.Numbers.Cyclic.Int63.Cyclic63

-

Uint63 numbers defines indeed a cyclic structure : Z/(2^63)Z

+

Uint63 numbers defines indeed a cyclic structure : Z/(2^63)Z

diff --git a/master/stdlib/Stdlib.Numbers.Cyclic.Int63.Ring63.html b/master/stdlib/Stdlib.Numbers.Cyclic.Int63.Ring63.html index be221ee839..cd60778c65 100644 --- a/master/stdlib/Stdlib.Numbers.Cyclic.Int63.Ring63.html +++ b/master/stdlib/Stdlib.Numbers.Cyclic.Int63.Ring63.html @@ -49,7 +49,7 @@

Library Stdlib.Numbers.Cyclic.Int63.Ring63

-

Uint63 numbers defines Z/(2^63)Z, and can hence be equipped

+

Uint63 numbers defines Z/(2^63)Z, and can hence be equipped

with a ring structure and a ring tactic
diff --git a/master/stdlib/Stdlib.Numbers.DecimalFacts.html b/master/stdlib/Stdlib.Numbers.DecimalFacts.html index 4f9ac1b3c7..1ecabfc6bd 100644 --- a/master/stdlib/Stdlib.Numbers.DecimalFacts.html +++ b/master/stdlib/Stdlib.Numbers.DecimalFacts.html @@ -49,7 +49,7 @@

Library Stdlib.Numbers.DecimalFacts

-

DecimalFacts : some facts about Decimal numbers

+

DecimalFacts : some facts about Decimal numbers

diff --git a/master/stdlib/Stdlib.Numbers.DecimalN.html b/master/stdlib/Stdlib.Numbers.DecimalN.html index 2398e9298b..d253f8e7cc 100644 --- a/master/stdlib/Stdlib.Numbers.DecimalN.html +++ b/master/stdlib/Stdlib.Numbers.DecimalN.html @@ -49,7 +49,7 @@

Library Stdlib.Numbers.DecimalN

-

DecimalN

+

DecimalN

diff --git a/master/stdlib/Stdlib.Numbers.DecimalNat.html b/master/stdlib/Stdlib.Numbers.DecimalNat.html index 7240ce8222..10ebf28372 100644 --- a/master/stdlib/Stdlib.Numbers.DecimalNat.html +++ b/master/stdlib/Stdlib.Numbers.DecimalNat.html @@ -49,7 +49,7 @@

Library Stdlib.Numbers.DecimalNat

-

DecimalNat

+

DecimalNat

diff --git a/master/stdlib/Stdlib.Numbers.DecimalPos.html b/master/stdlib/Stdlib.Numbers.DecimalPos.html index 8f00978222..e02bb16195 100644 --- a/master/stdlib/Stdlib.Numbers.DecimalPos.html +++ b/master/stdlib/Stdlib.Numbers.DecimalPos.html @@ -49,7 +49,7 @@

Library Stdlib.Numbers.DecimalPos

-

DecimalPos

+

DecimalPos

diff --git a/master/stdlib/Stdlib.Numbers.DecimalQ.html b/master/stdlib/Stdlib.Numbers.DecimalQ.html index 127a4759c9..57dd0d7aeb 100644 --- a/master/stdlib/Stdlib.Numbers.DecimalQ.html +++ b/master/stdlib/Stdlib.Numbers.DecimalQ.html @@ -49,7 +49,7 @@

Library Stdlib.Numbers.DecimalQ

-

DecimalQ

+

DecimalQ

diff --git a/master/stdlib/Stdlib.Numbers.DecimalR.html b/master/stdlib/Stdlib.Numbers.DecimalR.html index db543a6e4e..cb91aaebf2 100644 --- a/master/stdlib/Stdlib.Numbers.DecimalR.html +++ b/master/stdlib/Stdlib.Numbers.DecimalR.html @@ -49,7 +49,7 @@

Library Stdlib.Numbers.DecimalR

-

DecimalR

+

DecimalR

diff --git a/master/stdlib/Stdlib.Numbers.DecimalString.html b/master/stdlib/Stdlib.Numbers.DecimalString.html index e8646a99a1..8b8a343250 100644 --- a/master/stdlib/Stdlib.Numbers.DecimalString.html +++ b/master/stdlib/Stdlib.Numbers.DecimalString.html @@ -52,7 +52,7 @@

Library Stdlib.Numbers.DecimalString

-

Conversion between decimal numbers and Coq strings

+

Conversion between decimal numbers and Coq strings

diff --git a/master/stdlib/Stdlib.Numbers.DecimalZ.html b/master/stdlib/Stdlib.Numbers.DecimalZ.html index 1b19080f72..520a6c3011 100644 --- a/master/stdlib/Stdlib.Numbers.DecimalZ.html +++ b/master/stdlib/Stdlib.Numbers.DecimalZ.html @@ -49,7 +49,7 @@

Library Stdlib.Numbers.DecimalZ

-

DecimalZ

+

DecimalZ

diff --git a/master/stdlib/Stdlib.Numbers.HexadecimalFacts.html b/master/stdlib/Stdlib.Numbers.HexadecimalFacts.html index 843961f1f5..de885036e6 100644 --- a/master/stdlib/Stdlib.Numbers.HexadecimalFacts.html +++ b/master/stdlib/Stdlib.Numbers.HexadecimalFacts.html @@ -49,7 +49,7 @@

Library Stdlib.Numbers.HexadecimalFacts

-

HexadecimalFacts : some facts about Hexadecimal numbers

+

HexadecimalFacts : some facts about Hexadecimal numbers

diff --git a/master/stdlib/Stdlib.Numbers.HexadecimalN.html b/master/stdlib/Stdlib.Numbers.HexadecimalN.html index 7d1c5ec548..4fe08075a9 100644 --- a/master/stdlib/Stdlib.Numbers.HexadecimalN.html +++ b/master/stdlib/Stdlib.Numbers.HexadecimalN.html @@ -49,7 +49,7 @@

Library Stdlib.Numbers.HexadecimalN

-

HexadecimalN

+

HexadecimalN

diff --git a/master/stdlib/Stdlib.Numbers.HexadecimalNat.html b/master/stdlib/Stdlib.Numbers.HexadecimalNat.html index 3962d1f47c..4d78a09134 100644 --- a/master/stdlib/Stdlib.Numbers.HexadecimalNat.html +++ b/master/stdlib/Stdlib.Numbers.HexadecimalNat.html @@ -49,7 +49,7 @@

Library Stdlib.Numbers.HexadecimalNat

-

HexadecimalNat

+

HexadecimalNat

diff --git a/master/stdlib/Stdlib.Numbers.HexadecimalPos.html b/master/stdlib/Stdlib.Numbers.HexadecimalPos.html index 9ceb09926f..0a7fdffac7 100644 --- a/master/stdlib/Stdlib.Numbers.HexadecimalPos.html +++ b/master/stdlib/Stdlib.Numbers.HexadecimalPos.html @@ -49,7 +49,7 @@

Library Stdlib.Numbers.HexadecimalPos

-

HexadecimalPos

+

HexadecimalPos

diff --git a/master/stdlib/Stdlib.Numbers.HexadecimalQ.html b/master/stdlib/Stdlib.Numbers.HexadecimalQ.html index 5c8ce9a044..5ae7290d8b 100644 --- a/master/stdlib/Stdlib.Numbers.HexadecimalQ.html +++ b/master/stdlib/Stdlib.Numbers.HexadecimalQ.html @@ -49,7 +49,7 @@

Library Stdlib.Numbers.HexadecimalQ

-

HexadecimalQ

+

HexadecimalQ

diff --git a/master/stdlib/Stdlib.Numbers.HexadecimalR.html b/master/stdlib/Stdlib.Numbers.HexadecimalR.html index 9fb41d0066..bfb77f5e39 100644 --- a/master/stdlib/Stdlib.Numbers.HexadecimalR.html +++ b/master/stdlib/Stdlib.Numbers.HexadecimalR.html @@ -49,7 +49,7 @@

Library Stdlib.Numbers.HexadecimalR

-

HexadecimalR

+

HexadecimalR

diff --git a/master/stdlib/Stdlib.Numbers.HexadecimalString.html b/master/stdlib/Stdlib.Numbers.HexadecimalString.html index aaec98d61e..3cf7e19266 100644 --- a/master/stdlib/Stdlib.Numbers.HexadecimalString.html +++ b/master/stdlib/Stdlib.Numbers.HexadecimalString.html @@ -52,7 +52,7 @@

Library Stdlib.Numbers.HexadecimalString

-

Conversion between hexadecimal numbers and Coq strings

+

Conversion between hexadecimal numbers and Coq strings

diff --git a/master/stdlib/Stdlib.Numbers.HexadecimalZ.html b/master/stdlib/Stdlib.Numbers.HexadecimalZ.html index efb73cde60..4a3a781c6e 100644 --- a/master/stdlib/Stdlib.Numbers.HexadecimalZ.html +++ b/master/stdlib/Stdlib.Numbers.HexadecimalZ.html @@ -49,7 +49,7 @@

Library Stdlib.Numbers.HexadecimalZ

-

HexadecimalZ

+

HexadecimalZ

diff --git a/master/stdlib/Stdlib.Numbers.Integer.Abstract.ZBits.html b/master/stdlib/Stdlib.Numbers.Integer.Abstract.ZBits.html index 87a45d9a04..6078209f1b 100644 --- a/master/stdlib/Stdlib.Numbers.Integer.Abstract.ZBits.html +++ b/master/stdlib/Stdlib.Numbers.Integer.Abstract.ZBits.html @@ -473,7 +473,7 @@

Library Stdlib.Numbers.Integer.Abstract.ZBits

-

Properties of shifts

+

Properties of shifts

diff --git a/master/stdlib/Stdlib.Numbers.Integer.Abstract.ZDivEucl.html b/master/stdlib/Stdlib.Numbers.Integer.Abstract.ZDivEucl.html index d5e694926d..1018bac41c 100644 --- a/master/stdlib/Stdlib.Numbers.Integer.Abstract.ZDivEucl.html +++ b/master/stdlib/Stdlib.Numbers.Integer.Abstract.ZDivEucl.html @@ -55,7 +55,7 @@

Library Stdlib.Numbers.Integer.Abstract.ZDivEucl

-

Euclidean Division for integers, Euclid convention

+

Euclidean Division for integers, Euclid convention

@@ -246,7 +246,7 @@

Library Stdlib.Numbers.Integer.Abstract.ZDivEucl

-

Basic values of divisions and modulo.

+

Basic values of divisions and modulo.

@@ -282,7 +282,7 @@

Library Stdlib.Numbers.Integer.Abstract.ZDivEucl

-

Order results about mod and div

+

Order results about mod and div

@@ -411,7 +411,7 @@

Library Stdlib.Numbers.Integer.Abstract.ZDivEucl

-

Relations between usual operations and mod and div

+

Relations between usual operations and mod and div

diff --git a/master/stdlib/Stdlib.Numbers.Integer.Abstract.ZDivFloor.html b/master/stdlib/Stdlib.Numbers.Integer.Abstract.ZDivFloor.html index d01bfd4a68..c946bd0287 100644 --- a/master/stdlib/Stdlib.Numbers.Integer.Abstract.ZDivFloor.html +++ b/master/stdlib/Stdlib.Numbers.Integer.Abstract.ZDivFloor.html @@ -52,7 +52,7 @@

Library Stdlib.Numbers.Integer.Abstract.ZDivFloor

-

Euclidean Division for integers (Floor convention)

+

Euclidean Division for integers (Floor convention)

@@ -284,7 +284,7 @@

Library Stdlib.Numbers.Integer.Abstract.ZDivFloor

-

Basic values of divisions and modulo.

+

Basic values of divisions and modulo.

@@ -320,7 +320,7 @@

Library Stdlib.Numbers.Integer.Abstract.ZDivFloor

-

Order results about mod and div

+

Order results about mod and div

@@ -457,7 +457,7 @@

Library Stdlib.Numbers.Integer.Abstract.ZDivFloor

-

Relations between usual operations and mod and div

+

Relations between usual operations and mod and div

diff --git a/master/stdlib/Stdlib.Numbers.Integer.Abstract.ZDivTrunc.html b/master/stdlib/Stdlib.Numbers.Integer.Abstract.ZDivTrunc.html index ee9e76839d..fe9533bea1 100644 --- a/master/stdlib/Stdlib.Numbers.Integer.Abstract.ZDivTrunc.html +++ b/master/stdlib/Stdlib.Numbers.Integer.Abstract.ZDivTrunc.html @@ -52,7 +52,7 @@

Library Stdlib.Numbers.Integer.Abstract.ZDivTrunc

-

Euclidean Division for integers (Trunc convention)

+

Euclidean Division for integers (Trunc convention)

@@ -209,7 +209,7 @@

Library Stdlib.Numbers.Integer.Abstract.ZDivTrunc

-

Basic values of divisions and modulo.

+

Basic values of divisions and modulo.

@@ -307,7 +307,7 @@

Library Stdlib.Numbers.Integer.Abstract.ZDivTrunc

-

Order results about rem and quot

+

Order results about rem and quot

@@ -442,7 +442,7 @@

Library Stdlib.Numbers.Integer.Abstract.ZDivTrunc

-

Relations between usual operations and rem and quot

+

Relations between usual operations and rem and quot

diff --git a/master/stdlib/Stdlib.Numbers.Integer.Abstract.ZLcm.html b/master/stdlib/Stdlib.Numbers.Integer.Abstract.ZLcm.html index 2cd28f311b..9a6cea1c89 100644 --- a/master/stdlib/Stdlib.Numbers.Integer.Abstract.ZLcm.html +++ b/master/stdlib/Stdlib.Numbers.Integer.Abstract.ZLcm.html @@ -52,7 +52,7 @@

Library Stdlib.Numbers.Integer.Abstract.ZLcm

-

Least Common Multiple

+

Least Common Multiple

diff --git a/master/stdlib/Stdlib.Numbers.Integer.Abstract.ZMaxMin.html b/master/stdlib/Stdlib.Numbers.Integer.Abstract.ZMaxMin.html index be4ec3aca3..46ad4e691c 100644 --- a/master/stdlib/Stdlib.Numbers.Integer.Abstract.ZMaxMin.html +++ b/master/stdlib/Stdlib.Numbers.Integer.Abstract.ZMaxMin.html @@ -52,7 +52,7 @@

Library Stdlib.Numbers.Integer.Abstract.ZMaxMin

-

Properties of minimum and maximum specific to integer numbers

+

Properties of minimum and maximum specific to integer numbers

diff --git a/master/stdlib/Stdlib.Numbers.Integer.Binary.ZBinary.html b/master/stdlib/Stdlib.Numbers.Integer.Binary.ZBinary.html index 6022498220..a12ee75c55 100644 --- a/master/stdlib/Stdlib.Numbers.Integer.Binary.ZBinary.html +++ b/master/stdlib/Stdlib.Numbers.Integer.Binary.ZBinary.html @@ -71,7 +71,7 @@

Library Stdlib.Numbers.Integer.Binary.ZBinary

-

An order tactic for integers

+

An order tactic for integers

diff --git a/master/stdlib/Stdlib.Numbers.NaryFunctions.html b/master/stdlib/Stdlib.Numbers.NaryFunctions.html index 1142cba176..3e05cb270b 100644 --- a/master/stdlib/Stdlib.Numbers.NaryFunctions.html +++ b/master/stdlib/Stdlib.Numbers.NaryFunctions.html @@ -57,7 +57,7 @@

Library Stdlib.Numbers.NaryFunctions

-

Generic dependently-typed operators about n-ary functions

+

Generic dependently-typed operators about n-ary functions

diff --git a/master/stdlib/Stdlib.Numbers.NatInt.NZAdd.html b/master/stdlib/Stdlib.Numbers.NatInt.NZAdd.html index f976c777ea..6910b457d0 100644 --- a/master/stdlib/Stdlib.Numbers.NatInt.NZAdd.html +++ b/master/stdlib/Stdlib.Numbers.NatInt.NZAdd.html @@ -49,7 +49,7 @@

Library Stdlib.Numbers.NatInt.NZAdd

-

Some properties of the addition for modules implementing NZBasicFunsSig'

+

Some properties of the addition for modules implementing NZBasicFunsSig'

diff --git a/master/stdlib/Stdlib.Numbers.NatInt.NZAddOrder.html b/master/stdlib/Stdlib.Numbers.NatInt.NZAddOrder.html index 8d9af2fdc5..aab95e4c0d 100644 --- a/master/stdlib/Stdlib.Numbers.NatInt.NZAddOrder.html +++ b/master/stdlib/Stdlib.Numbers.NatInt.NZAddOrder.html @@ -49,7 +49,7 @@

Library Stdlib.Numbers.NatInt.NZAddOrder

-

Properties of orders and addition for modules implementing NZOrdAxiomsSig'

+

Properties of orders and addition for modules implementing NZOrdAxiomsSig'

diff --git a/master/stdlib/Stdlib.Numbers.NatInt.NZAxioms.html b/master/stdlib/Stdlib.Numbers.NatInt.NZAxioms.html index de170c4a1c..2071dc5e04 100644 --- a/master/stdlib/Stdlib.Numbers.NatInt.NZAxioms.html +++ b/master/stdlib/Stdlib.Numbers.NatInt.NZAxioms.html @@ -52,7 +52,7 @@

Library Stdlib.Numbers.NatInt.NZAxioms

Initial Author : Evgeny Makarov, INRIA, 2007
-

Axioms for a domain with zero, succ, pred.

+

Axioms for a domain with zero, succ, pred.

@@ -145,7 +145,7 @@

Library Stdlib.Numbers.NatInt.NZAxioms

-

Axiomatization of a domain with zero, succ, pred and a bi-directional induction principle.

+

Axiomatization of a domain with zero, succ, pred and a bi-directional induction principle.

@@ -227,7 +227,7 @@

Library Stdlib.Numbers.NatInt.NZAxioms

-

Axiomatization of some more constants

+

Axiomatization of some more constants

@@ -284,7 +284,7 @@

Library Stdlib.Numbers.NatInt.NZAxioms

-

Axiomatization of basic operations : + - *

+

Axiomatization of basic operations : + - *

@@ -340,7 +340,7 @@

Library Stdlib.Numbers.NatInt.NZAxioms

-

Axiomatization of order

+

Axiomatization of order

diff --git a/master/stdlib/Stdlib.Numbers.NatInt.NZBase.html b/master/stdlib/Stdlib.Numbers.NatInt.NZBase.html index d9474acc15..bb1b588790 100644 --- a/master/stdlib/Stdlib.Numbers.NatInt.NZBase.html +++ b/master/stdlib/Stdlib.Numbers.NatInt.NZBase.html @@ -49,7 +49,7 @@

Library Stdlib.Numbers.NatInt.NZBase

-

Basic lemmas about modules implementing NZDomainSig'

+

Basic lemmas about modules implementing NZDomainSig'

diff --git a/master/stdlib/Stdlib.Numbers.NatInt.NZDiv.html b/master/stdlib/Stdlib.Numbers.NatInt.NZDiv.html index d21aa69855..8beddeb790 100644 --- a/master/stdlib/Stdlib.Numbers.NatInt.NZDiv.html +++ b/master/stdlib/Stdlib.Numbers.NatInt.NZDiv.html @@ -190,7 +190,7 @@

Library Stdlib.Numbers.NatInt.NZDiv

-

Basic values of divisions and modulo.

+

Basic values of divisions and modulo.

@@ -223,7 +223,7 @@

Library Stdlib.Numbers.NatInt.NZDiv

-

Order results about mod and div

+

Order results about mod and div

@@ -335,7 +335,7 @@

Library Stdlib.Numbers.NatInt.NZDiv

-

Relations between usual operations and mod and div

+

Relations between usual operations and mod and div

diff --git a/master/stdlib/Stdlib.Numbers.NatInt.NZDomain.html b/master/stdlib/Stdlib.Numbers.NatInt.NZDomain.html index 3af3e4181e..266a5fde7a 100644 --- a/master/stdlib/Stdlib.Numbers.NatInt.NZDomain.html +++ b/master/stdlib/Stdlib.Numbers.NatInt.NZDomain.html @@ -78,7 +78,7 @@

Library Stdlib.Numbers.NatInt.NZDomain

-

Relationship between points thanks to succ and pred.

+

Relationship between points thanks to succ and pred.

@@ -129,7 +129,7 @@

Library Stdlib.Numbers.NatInt.NZDomain

-

Study of initial point w.r.t. succ (if any).

+

Study of initial point w.r.t. succ (if any).

@@ -253,7 +253,7 @@

Library Stdlib.Numbers.NatInt.NZDomain

-

An alternative induction principle using S and P.

+

An alternative induction principle using S and P.

diff --git a/master/stdlib/Stdlib.Numbers.NatInt.NZLog.html b/master/stdlib/Stdlib.Numbers.NatInt.NZLog.html index 36e45a37ba..37a0e638f5 100644 --- a/master/stdlib/Stdlib.Numbers.NatInt.NZLog.html +++ b/master/stdlib/Stdlib.Numbers.NatInt.NZLog.html @@ -418,7 +418,7 @@

Library Stdlib.Numbers.NatInt.NZLog

-

log2_up : a binary logarithm that rounds up instead of down

+

log2_up : a binary logarithm that rounds up instead of down

diff --git a/master/stdlib/Stdlib.Numbers.NatInt.NZMul.html b/master/stdlib/Stdlib.Numbers.NatInt.NZMul.html index 2f148f3343..7d05539c3f 100644 --- a/master/stdlib/Stdlib.Numbers.NatInt.NZMul.html +++ b/master/stdlib/Stdlib.Numbers.NatInt.NZMul.html @@ -49,7 +49,7 @@

Library Stdlib.Numbers.NatInt.NZMul

-

Some properties of the multiplication for modules implementing NZBasicFunsSig'

+

Some properties of the multiplication for modules implementing NZBasicFunsSig'

diff --git a/master/stdlib/Stdlib.Numbers.NatInt.NZMulOrder.html b/master/stdlib/Stdlib.Numbers.NatInt.NZMulOrder.html index 3394d6bc94..e5ac929473 100644 --- a/master/stdlib/Stdlib.Numbers.NatInt.NZMulOrder.html +++ b/master/stdlib/Stdlib.Numbers.NatInt.NZMulOrder.html @@ -49,7 +49,7 @@

Library Stdlib.Numbers.NatInt.NZMulOrder

-

Properties of orders and multiplication for modules implementing NZOrdAxiomsSig'

+

Properties of orders and multiplication for modules implementing NZOrdAxiomsSig'

diff --git a/master/stdlib/Stdlib.Numbers.NatInt.NZOrder.html b/master/stdlib/Stdlib.Numbers.NatInt.NZOrder.html index bde5d9905c..9b91b16972 100644 --- a/master/stdlib/Stdlib.Numbers.NatInt.NZOrder.html +++ b/master/stdlib/Stdlib.Numbers.NatInt.NZOrder.html @@ -49,7 +49,7 @@

Library Stdlib.Numbers.NatInt.NZOrder

-

Lemmas about orders for modules implementing NZOrdSig'

+

Lemmas about orders for modules implementing NZOrdSig'

@@ -105,11 +105,11 @@

Library Stdlib.Numbers.NatInt.NZOrder

-

Basic facts about le, lt, eq and succ

+

Basic facts about le, lt, eq and succ

-

Direct consequences of the specifications of lt and le

+

Direct consequences of the specifications of lt and le

@@ -167,7 +167,7 @@

Library Stdlib.Numbers.NatInt.NZOrder

-

Asymmetry and transitivity.

+

Asymmetry and transitivity.

@@ -188,7 +188,7 @@

Library Stdlib.Numbers.NatInt.NZOrder

-

Some type classes about order

+

Some type classes about order

@@ -209,7 +209,7 @@

Library Stdlib.Numbers.NatInt.NZOrder

-

Making the generic order tactic

+

Making the generic order tactic

@@ -236,7 +236,7 @@

Library Stdlib.Numbers.NatInt.NZOrder

-

Some direct consequences of order

+

Some direct consequences of order

@@ -281,7 +281,7 @@

Library Stdlib.Numbers.NatInt.NZOrder

-

More properties of < and <= with respect to S and 0

+

More properties of < and <= with respect to S and 0

@@ -337,7 +337,7 @@

Library Stdlib.Numbers.NatInt.NZOrder

-

More Trichotomy, decidability and double negation elimination

+

More Trichotomy, decidability and double negation elimination

@@ -448,7 +448,7 @@

Library Stdlib.Numbers.NatInt.NZOrder

-

Order-based induction principles

+

Order-based induction principles

diff --git a/master/stdlib/Stdlib.Numbers.NatInt.NZSqrt.html b/master/stdlib/Stdlib.Numbers.NatInt.NZSqrt.html index 3d397e7e9a..24f1ecb096 100644 --- a/master/stdlib/Stdlib.Numbers.NatInt.NZSqrt.html +++ b/master/stdlib/Stdlib.Numbers.NatInt.NZSqrt.html @@ -348,7 +348,7 @@

Library Stdlib.Numbers.NatInt.NZSqrt

-

sqrt_up : a square root that rounds up instead of down

+

sqrt_up : a square root that rounds up instead of down

diff --git a/master/stdlib/Stdlib.Numbers.Natural.Abstract.NDiv.html b/master/stdlib/Stdlib.Numbers.Natural.Abstract.NDiv.html index deb1e34cb2..051fecdc51 100644 --- a/master/stdlib/Stdlib.Numbers.Natural.Abstract.NDiv.html +++ b/master/stdlib/Stdlib.Numbers.Natural.Abstract.NDiv.html @@ -158,7 +158,7 @@

Library Stdlib.Numbers.Natural.Abstract.NDiv

-

Basic values of divisions and modulo.

+

Basic values of divisions and modulo.

@@ -191,7 +191,7 @@

Library Stdlib.Numbers.Natural.Abstract.NDiv

-

Order results about mod and div

+

Order results about mod and div

@@ -289,7 +289,7 @@

Library Stdlib.Numbers.Natural.Abstract.NDiv

-

Relations between usual operations and mod and div

+

Relations between usual operations and mod and div

diff --git a/master/stdlib/Stdlib.Numbers.Natural.Abstract.NLcm.html b/master/stdlib/Stdlib.Numbers.Natural.Abstract.NLcm.html index 21aa77837d..9f9ec15a51 100644 --- a/master/stdlib/Stdlib.Numbers.Natural.Abstract.NLcm.html +++ b/master/stdlib/Stdlib.Numbers.Natural.Abstract.NLcm.html @@ -52,7 +52,7 @@

Library Stdlib.Numbers.Natural.Abstract.NLcm

-

Least Common Multiple

+

Least Common Multiple

diff --git a/master/stdlib/Stdlib.Numbers.Natural.Abstract.NMaxMin.html b/master/stdlib/Stdlib.Numbers.Natural.Abstract.NMaxMin.html index b147831bec..ba18664e81 100644 --- a/master/stdlib/Stdlib.Numbers.Natural.Abstract.NMaxMin.html +++ b/master/stdlib/Stdlib.Numbers.Natural.Abstract.NMaxMin.html @@ -52,7 +52,7 @@

Library Stdlib.Numbers.Natural.Abstract.NMaxMin

-

Properties of minimum and maximum specific to natural numbers

+

Properties of minimum and maximum specific to natural numbers

diff --git a/master/stdlib/Stdlib.Numbers.Natural.Binary.NBinary.html b/master/stdlib/Stdlib.Numbers.Natural.Binary.NBinary.html index ee7685fced..14ccab9e43 100644 --- a/master/stdlib/Stdlib.Numbers.Natural.Binary.NBinary.html +++ b/master/stdlib/Stdlib.Numbers.Natural.Binary.NBinary.html @@ -59,7 +59,7 @@

Library Stdlib.Numbers.Natural.Binary.NBinary

-

BinNat.N already implements NAxiomSig

+

BinNat.N already implements NAxiomSig

diff --git a/master/stdlib/Stdlib.PArith.BinPos.html b/master/stdlib/Stdlib.PArith.BinPos.html index bc81b07cfa..0667072005 100644 --- a/master/stdlib/Stdlib.PArith.BinPos.html +++ b/master/stdlib/Stdlib.PArith.BinPos.html @@ -57,7 +57,7 @@

Library Stdlib.PArith.BinPos

-

Binary positive numbers, operations and properties

+

Binary positive numbers, operations and properties

@@ -91,7 +91,7 @@

Library Stdlib.PArith.BinPos

-

Definitions of operations, now in a separate file

+

Definitions of operations, now in a separate file

@@ -113,7 +113,7 @@

Library Stdlib.PArith.BinPos

-

Logical Predicates

+

Logical Predicates

@@ -145,11 +145,11 @@

Library Stdlib.PArith.BinPos

-

Properties of operations over positive numbers

+

Properties of operations over positive numbers

-

Decidability of equality on binary positive numbers

+

Decidability of equality on binary positive numbers

@@ -161,11 +161,11 @@

Library Stdlib.PArith.BinPos

-

Properties of successor on binary positive numbers

+

Properties of successor on binary positive numbers

-

Specification of xI in term of succ and xO

+

Specification of xI in term of succ and xO

@@ -180,7 +180,7 @@

Library Stdlib.PArith.BinPos

-

Successor and double

+

Successor and double

@@ -204,7 +204,7 @@

Library Stdlib.PArith.BinPos

-

Successor and predecessor

+

Successor and predecessor

@@ -225,7 +225,7 @@

Library Stdlib.PArith.BinPos

-

Injectivity of successor

+

Injectivity of successor

@@ -237,7 +237,7 @@

Library Stdlib.PArith.BinPos

-

Predecessor to N

+

Predecessor to N

@@ -249,11 +249,11 @@

Library Stdlib.PArith.BinPos

-

Properties of addition on binary positive numbers

+

Properties of addition on binary positive numbers

-

Specification of succ in term of add

+

Specification of succ in term of add

@@ -268,7 +268,7 @@

Library Stdlib.PArith.BinPos

-

Specification of add_carry

+

Specification of add_carry

@@ -280,7 +280,7 @@

Library Stdlib.PArith.BinPos

-

Commutativity

+

Commutativity

@@ -292,7 +292,7 @@

Library Stdlib.PArith.BinPos

-

Permutation of add and succ

+

Permutation of add and succ

@@ -307,7 +307,7 @@

Library Stdlib.PArith.BinPos

-

No neutral elements for addition

+

No neutral elements for addition

@@ -317,7 +317,7 @@

Library Stdlib.PArith.BinPos

-

Simplification

+

Simplification

@@ -350,7 +350,7 @@

Library Stdlib.PArith.BinPos

-

Addition is associative

+

Addition is associative

@@ -362,7 +362,7 @@

Library Stdlib.PArith.BinPos

-

Commutation of addition and double

+

Commutation of addition and double

@@ -382,7 +382,7 @@

Library Stdlib.PArith.BinPos

-

Miscellaneous

+

Miscellaneous

@@ -394,7 +394,7 @@

Library Stdlib.PArith.BinPos

-

Peano induction and recursion on binary positive positive numbers

+

Peano induction and recursion on binary positive positive numbers

@@ -512,11 +512,11 @@

Library Stdlib.PArith.BinPos

-

Properties of multiplication on binary positive numbers

+

Properties of multiplication on binary positive numbers

-

One is neutral for multiplication

+

One is neutral for multiplication

@@ -531,7 +531,7 @@

Library Stdlib.PArith.BinPos

-

Right reduction properties for multiplication

+

Right reduction properties for multiplication

@@ -546,7 +546,7 @@

Library Stdlib.PArith.BinPos

-

Commutativity of multiplication

+

Commutativity of multiplication

@@ -558,7 +558,7 @@

Library Stdlib.PArith.BinPos

-

Distributivity of multiplication over addition

+

Distributivity of multiplication over addition

@@ -575,7 +575,7 @@

Library Stdlib.PArith.BinPos

-

Associativity of multiplication

+

Associativity of multiplication

@@ -587,7 +587,7 @@

Library Stdlib.PArith.BinPos

-

Successor and multiplication

+

Successor and multiplication

@@ -602,7 +602,7 @@

Library Stdlib.PArith.BinPos

-

Parity properties of multiplication

+

Parity properties of multiplication

@@ -617,7 +617,7 @@

Library Stdlib.PArith.BinPos

-

Simplification properties of multiplication

+

Simplification properties of multiplication

@@ -638,7 +638,7 @@

Library Stdlib.PArith.BinPos

-

Inversion of multiplication

+

Inversion of multiplication

@@ -656,7 +656,7 @@

Library Stdlib.PArith.BinPos

-

Square

+

Square

@@ -671,7 +671,7 @@

Library Stdlib.PArith.BinPos

-

Properties of iter

+

Properties of iter

@@ -717,7 +717,7 @@

Library Stdlib.PArith.BinPos

-

Properties of power

+

Properties of power

@@ -732,7 +732,7 @@

Library Stdlib.PArith.BinPos

-

Properties of square

+

Properties of square

@@ -744,7 +744,7 @@

Library Stdlib.PArith.BinPos

-

Properties of sub_mask

+

Properties of sub_mask

@@ -791,7 +791,7 @@

Library Stdlib.PArith.BinPos

-

Properties of boolean comparisons

+

Properties of boolean comparisons

@@ -820,7 +820,7 @@

Library Stdlib.PArith.BinPos

-

Properties of comparison on binary positive numbers

+

Properties of comparison on binary positive numbers

@@ -1014,7 +1014,7 @@

Library Stdlib.PArith.BinPos

-

Facts about gt and ge

+

Facts about gt and ge

@@ -1047,7 +1047,7 @@

Library Stdlib.PArith.BinPos

-

Comparison and the successor

+

Comparison and the successor

@@ -1073,7 +1073,7 @@

Library Stdlib.PArith.BinPos

-

1 is the least positive number

+

1 is the least positive number

@@ -1091,7 +1091,7 @@

Library Stdlib.PArith.BinPos

-

Properties of the order

+

Properties of the order

@@ -1164,7 +1164,7 @@

Library Stdlib.PArith.BinPos

-

Comparison and addition

+

Comparison and addition

@@ -1179,7 +1179,7 @@

Library Stdlib.PArith.BinPos

-

Order and addition

+

Order and addition

@@ -1209,7 +1209,7 @@

Library Stdlib.PArith.BinPos

-

Comparison and multiplication

+

Comparison and multiplication

@@ -1224,7 +1224,7 @@

Library Stdlib.PArith.BinPos

-

Order and multiplication

+

Order and multiplication

@@ -1260,7 +1260,7 @@

Library Stdlib.PArith.BinPos

-

Properties of subtraction on binary positive numbers

+

Properties of subtraction on binary positive numbers

@@ -1278,7 +1278,7 @@

Library Stdlib.PArith.BinPos

-

Properties of subtraction without underflow

+

Properties of subtraction without underflow

@@ -1376,7 +1376,7 @@

Library Stdlib.PArith.BinPos

-

Results concerning size and size_nat

+

Results concerning size and size_nat

@@ -1394,7 +1394,7 @@

Library Stdlib.PArith.BinPos

-

Properties of min and max

+

Properties of min and max

@@ -1490,7 +1490,7 @@

Library Stdlib.PArith.BinPos

-

Results concerning iter_op

+

Results concerning iter_op

@@ -1511,7 +1511,7 @@

Library Stdlib.PArith.BinPos

-

Results about of_nat and of_succ_nat

+

Results about of_nat and of_succ_nat

@@ -1529,7 +1529,7 @@

Library Stdlib.PArith.BinPos

-

Correctness proofs for the square root function

+

Correctness proofs for the square root function

@@ -1555,7 +1555,7 @@

Library Stdlib.PArith.BinPos

-

Correctness proofs for the gcd function

+

Correctness proofs for the gcd function

diff --git a/master/stdlib/Stdlib.PArith.BinPosDef.html b/master/stdlib/Stdlib.PArith.BinPosDef.html index 93b60d6a1c..29b25cf694 100644 --- a/master/stdlib/Stdlib.PArith.BinPosDef.html +++ b/master/stdlib/Stdlib.PArith.BinPosDef.html @@ -49,7 +49,7 @@

Library Stdlib.PArith.BinPosDef

-

Binary positive numbers, operations

+

Binary positive numbers, operations

@@ -98,11 +98,11 @@

Library Stdlib.PArith.BinPosDef

-

Operations over positive numbers

+

Operations over positive numbers

-

Successor

+

Successor

@@ -119,7 +119,7 @@

Library Stdlib.PArith.BinPosDef

-

Addition

+

Addition

@@ -158,7 +158,7 @@

Library Stdlib.PArith.BinPosDef

-

Operation x -> 2*x-1

+

Operation x -> 2*x-1

@@ -175,7 +175,7 @@

Library Stdlib.PArith.BinPosDef

-

Predecessor

+

Predecessor

@@ -192,7 +192,7 @@

Library Stdlib.PArith.BinPosDef

-

The predecessor of a positive number can be seen as a N

+

The predecessor of a positive number can be seen as a N

@@ -209,7 +209,7 @@

Library Stdlib.PArith.BinPosDef

-

An auxiliary type for subtraction

+

An auxiliary type for subtraction

@@ -224,7 +224,7 @@

Library Stdlib.PArith.BinPosDef

-

Operation x -> 2*x+1

+

Operation x -> 2*x+1

@@ -241,7 +241,7 @@

Library Stdlib.PArith.BinPosDef

-

Operation x -> 2*x

+

Operation x -> 2*x

@@ -258,7 +258,7 @@

Library Stdlib.PArith.BinPosDef

-

Operation x -> 2*x-2

+

Operation x -> 2*x-2

@@ -275,7 +275,7 @@

Library Stdlib.PArith.BinPosDef

-

Predecessor with mask

+

Predecessor with mask

@@ -293,7 +293,7 @@

Library Stdlib.PArith.BinPosDef

-

Subtraction, result as a mask

+

Subtraction, result as a mask

@@ -326,7 +326,7 @@

Library Stdlib.PArith.BinPosDef

-

Subtraction, result as a positive, returning 1 if x<=y

+

Subtraction, result as a positive, returning 1 if x<=y

@@ -345,7 +345,7 @@

Library Stdlib.PArith.BinPosDef

-

Multiplication

+

Multiplication

@@ -365,7 +365,7 @@

Library Stdlib.PArith.BinPosDef

-

Iteration over a positive number

+

Iteration over a positive number

@@ -382,7 +382,7 @@

Library Stdlib.PArith.BinPosDef

-

Power

+

Power

@@ -397,7 +397,7 @@

Library Stdlib.PArith.BinPosDef

-

Square

+

Square

@@ -414,7 +414,7 @@

Library Stdlib.PArith.BinPosDef

-

Division by 2 rounded below but for 1

+

Division by 2 rounded below but for 1

@@ -447,7 +447,7 @@

Library Stdlib.PArith.BinPosDef

-

Number of digits in a positive number

+

Number of digits in a positive number

@@ -480,7 +480,7 @@

Library Stdlib.PArith.BinPosDef

-

Comparison on binary positive numbers

+

Comparison on binary positive numbers

@@ -523,7 +523,7 @@

Library Stdlib.PArith.BinPosDef

-

Boolean equality and comparisons

+

Boolean equality and comparisons

@@ -554,7 +554,7 @@

Library Stdlib.PArith.BinPosDef

-

A Square Root function for positive numbers

+

A Square Root function for positive numbers

@@ -600,7 +600,7 @@

Library Stdlib.PArith.BinPosDef

-

Greatest Common Divisor

+

Greatest Common Divisor

@@ -875,7 +875,7 @@

Library Stdlib.PArith.BinPosDef

-

From binary positive numbers to Peano natural numbers

+

From binary positive numbers to Peano natural numbers

@@ -895,7 +895,7 @@

Library Stdlib.PArith.BinPosDef

-

From Peano natural numbers to binary positive numbers

+

From Peano natural numbers to binary positive numbers

@@ -924,7 +924,7 @@

Library Stdlib.PArith.BinPosDef

-

Conversion with a decimal representation for printing/parsing

+

Conversion with a decimal representation for printing/parsing

diff --git a/master/stdlib/Stdlib.PArith.POrderedType.html b/master/stdlib/Stdlib.PArith.POrderedType.html index 95c8cffa0f..5874ca5486 100644 --- a/master/stdlib/Stdlib.PArith.POrderedType.html +++ b/master/stdlib/Stdlib.PArith.POrderedType.html @@ -55,7 +55,7 @@

Library Stdlib.PArith.POrderedType

-

DecidableType structure for positive numbers

+

DecidableType structure for positive numbers

@@ -71,7 +71,7 @@

Library Stdlib.PArith.POrderedType

interfaces, such as DecidableType or EqualityType.
-

OrderedType structure for positive numbers

+

OrderedType structure for positive numbers

@@ -87,7 +87,7 @@

Library Stdlib.PArith.POrderedType

and a OrderedType (and also as a DecidableType).
-

An order tactic for positive numbers

+

An order tactic for positive numbers

diff --git a/master/stdlib/Stdlib.Program.Combinators.html b/master/stdlib/Stdlib.Program.Combinators.html index 10739f9365..42b4c52b36 100644 --- a/master/stdlib/Stdlib.Program.Combinators.html +++ b/master/stdlib/Stdlib.Program.Combinators.html @@ -47,7 +47,7 @@

Library Stdlib.Program.Combinators

-

Proofs about standard combinators, exports functional extensionality.

+

Proofs about standard combinators, exports functional extensionality.

diff --git a/master/stdlib/Stdlib.QArith.QArith_base.html b/master/stdlib/Stdlib.QArith.QArith_base.html index f713bad5c0..85956aa496 100644 --- a/master/stdlib/Stdlib.QArith.QArith_base.html +++ b/master/stdlib/Stdlib.QArith.QArith_base.html @@ -55,7 +55,7 @@

Library Stdlib.QArith.QArith_base

-

Definition of Q and basic properties

+

Definition of Q and basic properties

@@ -198,7 +198,7 @@

Library Stdlib.QArith.QArith_base

-

Properties of equality.

+

Properties of equality.

@@ -290,7 +290,7 @@

Library Stdlib.QArith.QArith_base

-

Addition, multiplication and opposite

+

Addition, multiplication and opposite

@@ -557,7 +557,7 @@

Library Stdlib.QArith.QArith_base

-

Setoid compatibility results

+

Setoid compatibility results

@@ -631,7 +631,7 @@

Library Stdlib.QArith.QArith_base

-

Properties of Qadd

+

Properties of Qadd

@@ -671,7 +671,7 @@

Library Stdlib.QArith.QArith_base

-

Properties of Qopp

+

Properties of Qopp

@@ -702,7 +702,7 @@

Library Stdlib.QArith.QArith_base

-

Properties of Qmult

+

Properties of Qmult

@@ -784,7 +784,7 @@

Library Stdlib.QArith.QArith_base

-

inject_Z is a ring homomorphism:

+

inject_Z is a ring homomorphism:

@@ -802,7 +802,7 @@

Library Stdlib.QArith.QArith_base

-

Inverse and division.

+

Inverse and division.

@@ -854,11 +854,11 @@

Library Stdlib.QArith.QArith_base

-

Reduction and construction of Q

+

Reduction and construction of Q

-

Removal/introduction of common factor in both numerator and denominator.

+

Removal/introduction of common factor in both numerator and denominator.

@@ -903,7 +903,7 @@

Library Stdlib.QArith.QArith_base

-

Construction of a new rational by multiplication with an integer or pure fraction

+

Construction of a new rational by multiplication with an integer or pure fraction

@@ -929,7 +929,7 @@

Library Stdlib.QArith.QArith_base

-

Properties of order upon Q.

+

Properties of order upon Q.

@@ -1043,7 +1043,7 @@

Library Stdlib.QArith.QArith_base

-

Some decidability results about orders.

+

Some decidability results about orders.

@@ -1061,7 +1061,7 @@

Library Stdlib.QArith.QArith_base

-

Compatibility of addition with order

+

Compatibility of addition with order

@@ -1114,7 +1114,7 @@

Library Stdlib.QArith.QArith_base

-

Compatibility of multiplication with order.

+

Compatibility of multiplication with order.

@@ -1173,7 +1173,7 @@

Library Stdlib.QArith.QArith_base

-

Compatibility of inversion and division with order

+

Compatibility of inversion and division with order

@@ -1224,7 +1224,7 @@

Library Stdlib.QArith.QArith_base

-

Rational to the n-th power

+

Rational to the n-th power

diff --git a/master/stdlib/Stdlib.QArith.QOrderedType.html b/master/stdlib/Stdlib.QArith.QOrderedType.html index 25fc446636..c12a2e1adf 100644 --- a/master/stdlib/Stdlib.QArith.QOrderedType.html +++ b/master/stdlib/Stdlib.QArith.QOrderedType.html @@ -55,7 +55,7 @@

Library Stdlib.QArith.QOrderedType

-

DecidableType structure for rational numbers

+

DecidableType structure for rational numbers

@@ -93,7 +93,7 @@

Library Stdlib.QArith.QOrderedType

interfaces, such as DecidableType or EqualityType.
-

OrderedType structure for rational numbers

+

OrderedType structure for rational numbers

@@ -124,7 +124,7 @@

Library Stdlib.QArith.QOrderedType

-

An order tactic for Q numbers

+

An order tactic for Q numbers

diff --git a/master/stdlib/Stdlib.QArith.Qcabs.html b/master/stdlib/Stdlib.QArith.Qcabs.html index be63acf16c..d37b33e5e1 100644 --- a/master/stdlib/Stdlib.QArith.Qcabs.html +++ b/master/stdlib/Stdlib.QArith.Qcabs.html @@ -49,7 +49,7 @@

Library Stdlib.QArith.Qcabs

-

An absolute value for normalized rational numbers.

+

An absolute value for normalized rational numbers.

diff --git a/master/stdlib/Stdlib.QArith.Qfield.html b/master/stdlib/Stdlib.QArith.Qfield.html index 676a22168b..7015f115dd 100644 --- a/master/stdlib/Stdlib.QArith.Qfield.html +++ b/master/stdlib/Stdlib.QArith.Qfield.html @@ -54,7 +54,7 @@

Library Stdlib.QArith.Qfield

-

field and ring tactics for rational numbers

+

field and ring tactics for rational numbers

diff --git a/master/stdlib/Stdlib.QArith.Qminmax.html b/master/stdlib/Stdlib.QArith.Qminmax.html index 2f85ec76a6..4ed0d14b1c 100644 --- a/master/stdlib/Stdlib.QArith.Qminmax.html +++ b/master/stdlib/Stdlib.QArith.Qminmax.html @@ -52,7 +52,7 @@

Library Stdlib.QArith.Qminmax

-

Maximum and Minimum of two rational numbers

+

Maximum and Minimum of two rational numbers

@@ -101,7 +101,7 @@

Library Stdlib.QArith.Qminmax

-

Properties specific to the Q domain

+

Properties specific to the Q domain

diff --git a/master/stdlib/Stdlib.QArith.Qpower.html b/master/stdlib/Stdlib.QArith.Qpower.html index 749514ca04..871eed9887 100644 --- a/master/stdlib/Stdlib.QArith.Qpower.html +++ b/master/stdlib/Stdlib.QArith.Qpower.html @@ -52,11 +52,11 @@

Library Stdlib.QArith.Qpower

-

Properties of Qpower_positive

+

Properties of Qpower_positive

-

Values of Qpower_positive for specific arguments

+

Values of Qpower_positive for specific arguments

@@ -71,7 +71,7 @@

Library Stdlib.QArith.Qpower

-

Relation of Qpower_positive to zero

+

Relation of Qpower_positive to zero

@@ -86,7 +86,7 @@

Library Stdlib.QArith.Qpower

-

Qpower_positive and multiplication, exponent subtraction

+

Qpower_positive and multiplication, exponent subtraction

@@ -101,7 +101,7 @@

Library Stdlib.QArith.Qpower

-

Qpower_positive and inversion, division, exponent subtraction

+

Qpower_positive and inversion, division, exponent subtraction

@@ -118,7 +118,7 @@

Library Stdlib.QArith.Qpower

-

Qpower and exponent multiplication

+

Qpower and exponent multiplication

@@ -131,7 +131,7 @@

Library Stdlib.QArith.Qpower

-

Qpower_positive decomposition

+

Qpower_positive decomposition

@@ -147,11 +147,11 @@

Library Stdlib.QArith.Qpower

-

Properties of Qpower

+

Properties of Qpower

-

Values of Qpower for specific arguments

+

Values of Qpower for specific arguments

@@ -174,7 +174,7 @@

Library Stdlib.QArith.Qpower

-

Relation of Qpower to zero

+

Relation of Qpower to zero

@@ -196,7 +196,7 @@

Library Stdlib.QArith.Qpower

-

Relation of Qpower to 1

+

Relation of Qpower to 1

@@ -221,7 +221,7 @@

Library Stdlib.QArith.Qpower

-

Qpower and multiplication, exponent addition

+

Qpower and multiplication, exponent addition

@@ -239,7 +239,7 @@

Library Stdlib.QArith.Qpower

-

Qpower and inversion, division, exponent subtraction

+

Qpower and inversion, division, exponent subtraction

@@ -272,7 +272,7 @@

Library Stdlib.QArith.Qpower

-

Qpower and exponent multiplication

+

Qpower and exponent multiplication

@@ -284,7 +284,7 @@

Library Stdlib.QArith.Qpower

-

Qpower decomposition

+

Qpower decomposition

@@ -305,7 +305,7 @@

Library Stdlib.QArith.Qpower

-

Compatibility of Qpower with relational operators

+

Compatibility of Qpower with relational operators

@@ -330,7 +330,7 @@

Library Stdlib.QArith.Qpower

-

Qpower and inject_Z

+

Qpower and inject_Z

@@ -342,7 +342,7 @@

Library Stdlib.QArith.Qpower

-

Square

+

Square

@@ -354,7 +354,7 @@

Library Stdlib.QArith.Qpower

-

Power of 2 positive upper bound

+

Power of 2 positive upper bound

diff --git a/master/stdlib/Stdlib.Reals.AltSeries.html b/master/stdlib/Stdlib.Reals.AltSeries.html index 9f11afa662..fbb048ab8a 100644 --- a/master/stdlib/Stdlib.Reals.AltSeries.html +++ b/master/stdlib/Stdlib.Reals.AltSeries.html @@ -58,7 +58,7 @@

Library Stdlib.Reals.AltSeries

-

Formalization of alternated series

+

Formalization of alternated series

@@ -121,7 +121,7 @@

Library Stdlib.Reals.AltSeries

-

Convergence of alternated series

+

Convergence of alternated series

@@ -143,7 +143,7 @@

Library Stdlib.Reals.AltSeries

-

Application : construction of PI

+

Application : construction of PI

diff --git a/master/stdlib/Stdlib.Reals.Cauchy.ConstructiveCauchyReals.html b/master/stdlib/Stdlib.Reals.Cauchy.ConstructiveCauchyReals.html index df073f9be0..23b5300982 100644 --- a/master/stdlib/Stdlib.Reals.Cauchy.ConstructiveCauchyReals.html +++ b/master/stdlib/Stdlib.Reals.Cauchy.ConstructiveCauchyReals.html @@ -408,7 +408,7 @@

Library Stdlib.Reals.Cauchy.ConstructiveCauchyReals

-

Algebraic operations

+

Algebraic operations

diff --git a/master/stdlib/Stdlib.Reals.Cauchy.ConstructiveCauchyRealsMult.html b/master/stdlib/Stdlib.Reals.Cauchy.ConstructiveCauchyRealsMult.html index f799eb5d5e..930172e60a 100644 --- a/master/stdlib/Stdlib.Reals.Cauchy.ConstructiveCauchyRealsMult.html +++ b/master/stdlib/Stdlib.Reals.Cauchy.ConstructiveCauchyRealsMult.html @@ -296,7 +296,7 @@

Library Stdlib.Reals.Cauchy.ConstructiveCauchyRealsMult

-

Field

+

Field

diff --git a/master/stdlib/Stdlib.Reals.Cauchy.QExtra.html b/master/stdlib/Stdlib.Reals.Cauchy.QExtra.html index a1a1b1a503..66aefb9e64 100644 --- a/master/stdlib/Stdlib.Reals.Cauchy.QExtra.html +++ b/master/stdlib/Stdlib.Reals.Cauchy.QExtra.html @@ -55,7 +55,7 @@

Library Stdlib.Reals.Cauchy.QExtra

-

Power of 2 open and closed upper and lower bounds for q : Q

+

Power of 2 open and closed upper and lower bounds for q : Q

@@ -96,7 +96,7 @@

Library Stdlib.Reals.Cauchy.QExtra

-

Power of two closed upper bound q <= 2^z

+

Power of two closed upper bound q <= 2^z

@@ -125,7 +125,7 @@

Library Stdlib.Reals.Cauchy.QExtra

-

Power of two open upper bound q < 2^z and Qabs q < 2^z

+

Power of two open upper bound q < 2^z and Qabs q < 2^z

@@ -171,7 +171,7 @@

Library Stdlib.Reals.Cauchy.QExtra

-

Power of 2 open lower bounds for 2^z < q and 2^z < Qabs q

+

Power of 2 open lower bounds for 2^z < q and 2^z < Qabs q

@@ -202,7 +202,7 @@

Library Stdlib.Reals.Cauchy.QExtra

-

Existential formulations of power of 2 lower and upper bounds

+

Existential formulations of power of 2 lower and upper bounds

diff --git a/master/stdlib/Stdlib.Reals.ClassicalDedekindReals.html b/master/stdlib/Stdlib.Reals.ClassicalDedekindReals.html index 23d96ae862..938d51a66c 100644 --- a/master/stdlib/Stdlib.Reals.ClassicalDedekindReals.html +++ b/master/stdlib/Stdlib.Reals.ClassicalDedekindReals.html @@ -63,7 +63,7 @@

Library Stdlib.Reals.ClassicalDedekindReals

-

Q Auxiliary Lemmas

+

Q Auxiliary Lemmas

@@ -86,11 +86,11 @@

Library Stdlib.Reals.ClassicalDedekindReals

-

Dedekind cuts

+

Dedekind cuts

-

Definition

+

Definition

@@ -132,7 +132,7 @@

Library Stdlib.Reals.ClassicalDedekindReals

-

Properties

+

Properties

@@ -164,11 +164,11 @@

Library Stdlib.Reals.ClassicalDedekindReals

-

Classical Dedekind reals

+

Classical Dedekind reals

-

Definition

+

Definition

@@ -181,7 +181,7 @@

Library Stdlib.Reals.ClassicalDedekindReals

-

Induction principle

+

Induction principle

@@ -195,11 +195,11 @@

Library Stdlib.Reals.ClassicalDedekindReals

-

Conversion to and from constructive Cauchy real CReal

+

Conversion to and from constructive Cauchy real CReal

-

Conversion from CReal to DReal

+

Conversion from CReal to DReal

@@ -218,7 +218,7 @@

Library Stdlib.Reals.ClassicalDedekindReals

-

Conversion from DReal to CReal

+

Conversion from DReal to CReal

@@ -269,7 +269,7 @@

Library Stdlib.Reals.ClassicalDedekindReals

-

Order for DReal

+

Order for DReal

diff --git a/master/stdlib/Stdlib.Reals.RIneq.html b/master/stdlib/Stdlib.Reals.RIneq.html index ca9c10a67b..c8069d71eb 100644 --- a/master/stdlib/Stdlib.Reals.RIneq.html +++ b/master/stdlib/Stdlib.Reals.RIneq.html @@ -49,7 +49,7 @@

Library Stdlib.Reals.RIneq

-

Basic lemmas for the classical real numbers

+

Basic lemmas for the classical real numbers

@@ -137,7 +137,7 @@

Library Stdlib.Reals.RIneq

-

Relation between orders and equality

+

Relation between orders and equality

@@ -227,7 +227,7 @@

Library Stdlib.Reals.RIneq

-

Strong decidable equality

+

Strong decidable equality

@@ -239,11 +239,11 @@

Library Stdlib.Reals.RIneq

-

Relating <, >, <= and >=

+

Relating <, >, <= and >=

-

Relating strict and large orders

+

Relating strict and large orders

@@ -348,7 +348,7 @@

Library Stdlib.Reals.RIneq

-

Asymmetry

+

Asymmetry

@@ -369,7 +369,7 @@

Library Stdlib.Reals.RIneq

-

Antisymmetry

+

Antisymmetry

@@ -398,7 +398,7 @@

Library Stdlib.Reals.RIneq

-

Compatibility with equality

+

Compatibility with equality

@@ -415,7 +415,7 @@

Library Stdlib.Reals.RIneq

-

Transitivity

+

Transitivity

@@ -458,7 +458,7 @@

Library Stdlib.Reals.RIneq

-

(Classical) decidability with sumbool types

+

(Classical) decidability with sumbool types

@@ -509,7 +509,7 @@

Library Stdlib.Reals.RIneq

-

Same theorems with disjunctions instead of sumbools

+

Same theorems with disjunctions instead of sumbools

@@ -563,7 +563,7 @@

Library Stdlib.Reals.RIneq

-

Addition

+

Addition

@@ -637,7 +637,7 @@

Library Stdlib.Reals.RIneq

-

Opposite

+

Opposite

@@ -679,7 +679,7 @@

Library Stdlib.Reals.RIneq

-

Multiplication

+

Multiplication

@@ -795,7 +795,7 @@

Library Stdlib.Reals.RIneq

-

Opposite and multiplication

+

Opposite and multiplication

@@ -823,7 +823,7 @@

Library Stdlib.Reals.RIneq

-

Subtraction

+

Subtraction

@@ -935,7 +935,7 @@

Library Stdlib.Reals.RIneq

-

Inverse

+

Inverse

@@ -989,7 +989,7 @@

Library Stdlib.Reals.RIneq

-

Square function

+

Square function

@@ -1011,11 +1011,11 @@

Library Stdlib.Reals.RIneq

-

Order and addition

+

Order and addition

-

Compatibility

+

Compatibility

@@ -1116,7 +1116,7 @@

Library Stdlib.Reals.RIneq

-

Cancellation

+

Cancellation

@@ -1168,7 +1168,7 @@

Library Stdlib.Reals.RIneq

-

Comparison of addition with left operand

+

Comparison of addition with left operand

@@ -1189,7 +1189,7 @@

Library Stdlib.Reals.RIneq

-

Sign of addition

+

Sign of addition

@@ -1222,11 +1222,11 @@

Library Stdlib.Reals.RIneq

-

Order and opposite

+

Order and opposite

-

Contravariant compatibility

+

Contravariant compatibility

@@ -1302,7 +1302,7 @@

Library Stdlib.Reals.RIneq

-

Cancellation

+

Cancellation

@@ -1327,7 +1327,7 @@

Library Stdlib.Reals.RIneq

-

Sign of opposite

+

Sign of opposite

@@ -1342,14 +1342,14 @@

Library Stdlib.Reals.RIneq

-

Order and multiplication

+

Order and multiplication

Remark: Rmult_lt_compat_l is in Raxioms.v
-

Covariant compatibility

+

Covariant compatibility

@@ -1420,7 +1420,7 @@

Library Stdlib.Reals.RIneq

-

Contravariant compatibility

+

Contravariant compatibility

@@ -1445,7 +1445,7 @@

Library Stdlib.Reals.RIneq

-

Sign of multiplication

+

Sign of multiplication

@@ -1480,7 +1480,7 @@

Library Stdlib.Reals.RIneq

-

Order and square function

+

Order and square function

@@ -1501,7 +1501,7 @@

Library Stdlib.Reals.RIneq

-

Zero is less than one

+

Zero is less than one

@@ -1518,7 +1518,7 @@

Library Stdlib.Reals.RIneq

-

Sign of inverse

+

Sign of inverse

@@ -1537,7 +1537,7 @@

Library Stdlib.Reals.RIneq

-

Cancellation in inequalities of products

+

Cancellation in inequalities of products

@@ -1564,7 +1564,7 @@

Library Stdlib.Reals.RIneq

-

Order and inverse

+

Order and inverse

@@ -1595,7 +1595,7 @@

Library Stdlib.Reals.RIneq

-

Sign of inverse

+

Sign of inverse

@@ -1610,7 +1610,7 @@

Library Stdlib.Reals.RIneq

-

Order and subtraction

+

Order and subtraction

@@ -1654,7 +1654,7 @@

Library Stdlib.Reals.RIneq

-

Division

+

Division

@@ -1754,7 +1754,7 @@

Library Stdlib.Reals.RIneq

-

Sign of division

+

Sign of division

@@ -1779,7 +1779,7 @@

Library Stdlib.Reals.RIneq

-

Miscellaneous

+

Miscellaneous

@@ -1833,7 +1833,7 @@

Library Stdlib.Reals.RIneq

-

Injection from nat to R

+

Injection from nat to R

@@ -1932,7 +1932,7 @@

Library Stdlib.Reals.RIneq

-

Injection from positive to R

+

Injection from positive to R

@@ -2013,7 +2013,7 @@

Library Stdlib.Reals.RIneq

-

Injection from Z to R

+

Injection from Z to R

@@ -2150,7 +2150,7 @@

Library Stdlib.Reals.RIneq

-

Definitions of new types

+

Definitions of new types

@@ -2177,7 +2177,7 @@

Library Stdlib.Reals.RIneq

-

A few common instances

+

A few common instances

@@ -2193,7 +2193,7 @@

Library Stdlib.Reals.RIneq

-

Compatibility

+

Compatibility

diff --git a/master/stdlib/Stdlib.Reals.ROrderedType.html b/master/stdlib/Stdlib.Reals.ROrderedType.html index 0c78aebd8b..6565c93fe0 100644 --- a/master/stdlib/Stdlib.Reals.ROrderedType.html +++ b/master/stdlib/Stdlib.Reals.ROrderedType.html @@ -55,7 +55,7 @@

Library Stdlib.Reals.ROrderedType

-

DecidableType structure for real numbers

+

DecidableType structure for real numbers

@@ -90,7 +90,7 @@

Library Stdlib.Reals.ROrderedType

and a DecidableTypeOrig.
-

OrderedType structure for binary integers

+

OrderedType structure for binary integers

@@ -138,7 +138,7 @@

Library Stdlib.Reals.ROrderedType

and a OrderedType (and also as a DecidableType).
-

An order tactic for real numbers

+

An order tactic for real numbers

diff --git a/master/stdlib/Stdlib.Reals.R_Ifp.html b/master/stdlib/Stdlib.Reals.R_Ifp.html index b0df9eeed0..8ac6190863 100644 --- a/master/stdlib/Stdlib.Reals.R_Ifp.html +++ b/master/stdlib/Stdlib.Reals.R_Ifp.html @@ -62,7 +62,7 @@

Library Stdlib.Reals.R_Ifp

-

Fractional part

+

Fractional part

@@ -97,7 +97,7 @@

Library Stdlib.Reals.R_Ifp

-

Properties

+

Properties

diff --git a/master/stdlib/Stdlib.Reals.R_sqrt.html b/master/stdlib/Stdlib.Reals.R_sqrt.html index cef9ec79ad..bae828fb9c 100644 --- a/master/stdlib/Stdlib.Reals.R_sqrt.html +++ b/master/stdlib/Stdlib.Reals.R_sqrt.html @@ -55,7 +55,7 @@

Library Stdlib.Reals.R_sqrt

-

Continuous extension of Rsqrt on R

+

Continuous extension of Rsqrt on R

@@ -196,7 +196,7 @@

Library Stdlib.Reals.R_sqrt

-

Resolution of a*X^2+b*X+c=0

+

Resolution of a*X^2+b*X+c=0

diff --git a/master/stdlib/Stdlib.Reals.Ranalysis1.html b/master/stdlib/Stdlib.Reals.Ranalysis1.html index 29cd2e123b..cee8374289 100644 --- a/master/stdlib/Stdlib.Reals.Ranalysis1.html +++ b/master/stdlib/Stdlib.Reals.Ranalysis1.html @@ -57,7 +57,7 @@

Library Stdlib.Reals.Ranalysis1

-

Basic operations on functions

+

Basic operations on functions

@@ -106,7 +106,7 @@

Library Stdlib.Reals.Ranalysis1

-

Variations of functions

+

Variations of functions

@@ -127,7 +127,7 @@

Library Stdlib.Reals.Ranalysis1

-

Definition of continuity as a limit

+

Definition of continuity as a limit

@@ -231,7 +231,7 @@

Library Stdlib.Reals.Ranalysis1

-

Derivative's definition using Landau's kernel

+

Derivative's definition using Landau's kernel

@@ -271,7 +271,7 @@

Library Stdlib.Reals.Ranalysis1

-

Class of differential functions

+

Class of differential functions

@@ -327,7 +327,7 @@

Library Stdlib.Reals.Ranalysis1

-

Equivalence of this definition with the one using limit concept

+

Equivalence of this definition with the one using limit concept

@@ -358,7 +358,7 @@

Library Stdlib.Reals.Ranalysis1

-

derivability -> continuity

+

derivability -> continuity

@@ -376,11 +376,11 @@

Library Stdlib.Reals.Ranalysis1

-

Main rules

+

Main rules

-

Rules for derivable_pt_lim (value of the derivative at a point)

+

Rules for derivable_pt_lim (value of the derivative at a point)

@@ -458,7 +458,7 @@

Library Stdlib.Reals.Ranalysis1

-

Rules for derivable_pt (derivability at a point)

+

Rules for derivable_pt (derivability at a point)

@@ -524,7 +524,7 @@

Library Stdlib.Reals.Ranalysis1

-

Rules for derivable (derivability on whole domain)

+

Rules for derivable (derivability on whole domain)

@@ -568,7 +568,7 @@

Library Stdlib.Reals.Ranalysis1

-

Rules for derive_pt (derivative function on whole domain)

+

Rules for derive_pt (derivative function on whole domain)

@@ -638,7 +638,7 @@

Library Stdlib.Reals.Ranalysis1

-

Definition and derivative of power function with natural number exponent

+

Definition and derivative of power function with natural number exponent

@@ -672,7 +672,7 @@

Library Stdlib.Reals.Ranalysis1

-

Irrelevance of derivability proof for derivative

+

Irrelevance of derivability proof for derivative

@@ -700,7 +700,7 @@

Library Stdlib.Reals.Ranalysis1

-

Local extremum's condition

+

Local extremum's condition

diff --git a/master/stdlib/Stdlib.Reals.Ranalysis5.html b/master/stdlib/Stdlib.Reals.Ranalysis5.html index 1277f97c89..2c35bbbb45 100644 --- a/master/stdlib/Stdlib.Reals.Ranalysis5.html +++ b/master/stdlib/Stdlib.Reals.Ranalysis5.html @@ -63,7 +63,7 @@

Library Stdlib.Reals.Ranalysis5

-

Preliminaries lemmas

+

Preliminaries lemmas

@@ -139,11 +139,11 @@

Library Stdlib.Reals.Ranalysis5

-

The derivative of a reciprocal function

+

The derivative of a reciprocal function

-

Continuity of the reciprocal function

+

Continuity of the reciprocal function

@@ -171,7 +171,7 @@

Library Stdlib.Reals.Ranalysis5

-

Derivability of the reciprocal function

+

Derivability of the reciprocal function

@@ -245,7 +245,7 @@

Library Stdlib.Reals.Ranalysis5

-

Value of the derivative of the reciprocal function

+

Value of the derivative of the reciprocal function

@@ -321,7 +321,7 @@

Library Stdlib.Reals.Ranalysis5

-

Existence of the derivative of a function which is the limit of a sequence of functions

+

Existence of the derivative of a function which is the limit of a sequence of functions

diff --git a/master/stdlib/Stdlib.Reals.Ratan.html b/master/stdlib/Stdlib.Reals.Ratan.html index f02eee6393..f569a2ced3 100644 --- a/master/stdlib/Stdlib.Reals.Ratan.html +++ b/master/stdlib/Stdlib.Reals.Ratan.html @@ -69,11 +69,11 @@

Library Stdlib.Reals.Ratan

-

Preliminaries

+

Preliminaries

-

Various generic lemmas which probably should go somewhere else

+

Various generic lemmas which probably should go somewhere else

@@ -121,11 +121,11 @@

Library Stdlib.Reals.Ratan

-

Properties of tangent

+

Properties of tangent

-

Derivative of tangent

+

Derivative of tangent

@@ -143,7 +143,7 @@

Library Stdlib.Reals.Ratan

-

Proof that tangent is a bijection

+

Proof that tangent is a bijection

@@ -193,11 +193,11 @@

Library Stdlib.Reals.Ratan

-

Definition of arctangent

+

Definition of arctangent

-

Definition of arctangent as the reciprocal function of tangent and proof of this status

+

Definition of arctangent as the reciprocal function of tangent and proof of this status

@@ -270,7 +270,7 @@

Library Stdlib.Reals.Ratan

-

Derivative of arctangent

+

Derivative of arctangent

@@ -287,7 +287,7 @@

Library Stdlib.Reals.Ratan

-

Definition of the arctangent function as the sum of the arctan power series

+

Definition of the arctangent function as the sum of the arctan power series

@@ -335,7 +335,7 @@

Library Stdlib.Reals.Ratan

-

Proof of the equivalence of the two definitions between -1 and 1

+

Proof of the equivalence of the two definitions between -1 and 1

@@ -474,7 +474,7 @@

Library Stdlib.Reals.Ratan

-

Relation between arctangent and sine and cosine

+

Relation between arctangent and sine and cosine

@@ -491,7 +491,7 @@

Library Stdlib.Reals.Ratan

-

Definition of arcsine based on arctangent

+

Definition of arcsine based on arctangent

@@ -509,7 +509,7 @@

Library Stdlib.Reals.Ratan

-

Relation between arcsin and arctangent

+

Relation between arcsin and arctangent

@@ -522,7 +522,7 @@

Library Stdlib.Reals.Ratan

-

arcsine of specific values

+

arcsine of specific values

@@ -544,7 +544,7 @@

Library Stdlib.Reals.Ratan

-

Bounds of arcsine

+

Bounds of arcsine

@@ -561,7 +561,7 @@

Library Stdlib.Reals.Ratan

-

arcsine is the left and right inverse of sine

+

arcsine is the left and right inverse of sine

@@ -578,7 +578,7 @@

Library Stdlib.Reals.Ratan

-

Relation between arcsin, cosine and tangent

+

Relation between arcsin, cosine and tangent

@@ -595,7 +595,7 @@

Library Stdlib.Reals.Ratan

-

Derivative of arcsine

+

Derivative of arcsine

@@ -612,7 +612,7 @@

Library Stdlib.Reals.Ratan

-

Definition of arccosine based on arctangent

+

Definition of arccosine based on arctangent

@@ -630,7 +630,7 @@

Library Stdlib.Reals.Ratan

-

Relation between arccosine, arcsine and arctangent

+

Relation between arccosine, arcsine and arctangent

@@ -651,7 +651,7 @@

Library Stdlib.Reals.Ratan

-

arccosine of specific values

+

arccosine of specific values

@@ -673,7 +673,7 @@

Library Stdlib.Reals.Ratan

-

Bounds of arccosine

+

Bounds of arccosine

@@ -690,7 +690,7 @@

Library Stdlib.Reals.Ratan

-

arccosine is the left and right inverse of cosine

+

arccosine is the left and right inverse of cosine

@@ -707,7 +707,7 @@

Library Stdlib.Reals.Ratan

-

Relation between arccosine, sine and tangent

+

Relation between arccosine, sine and tangent

@@ -724,7 +724,7 @@

Library Stdlib.Reals.Ratan

-

Derivative of arccosine

+

Derivative of arccosine

diff --git a/master/stdlib/Stdlib.Reals.Raxioms.html b/master/stdlib/Stdlib.Reals.Raxioms.html index 335f2b8f54..03f8646546 100644 --- a/master/stdlib/Stdlib.Reals.Raxioms.html +++ b/master/stdlib/Stdlib.Reals.Raxioms.html @@ -69,11 +69,11 @@

Library Stdlib.Reals.Raxioms

-

Field operations

+

Field operations

-

Addition

+

Addition

@@ -141,7 +141,7 @@

Library Stdlib.Reals.Raxioms

-

Multiplication

+

Multiplication

@@ -176,7 +176,7 @@

Library Stdlib.Reals.Raxioms

-

Distributivity

+

Distributivity

@@ -192,11 +192,11 @@

Library Stdlib.Reals.Raxioms

-

Order

+

Order

-

Lower

+

Lower

@@ -222,7 +222,7 @@

Library Stdlib.Reals.Raxioms

-

Injection from N to R

+

Injection from N to R

@@ -241,7 +241,7 @@

Library Stdlib.Reals.Raxioms

-

R Archimedean

+

R Archimedean

@@ -269,7 +269,7 @@

Library Stdlib.Reals.Raxioms

-

R Complete

+

R Complete

diff --git a/master/stdlib/Stdlib.Reals.Rbasic_fun.html b/master/stdlib/Stdlib.Reals.Rbasic_fun.html index 767456cd1c..ab97d34f28 100644 --- a/master/stdlib/Stdlib.Reals.Rbasic_fun.html +++ b/master/stdlib/Stdlib.Reals.Rbasic_fun.html @@ -65,7 +65,7 @@

Library Stdlib.Reals.Rbasic_fun

-

Rmin

+

Rmin

@@ -131,7 +131,7 @@

Library Stdlib.Reals.Rbasic_fun

-

Rmax

+

Rmax

@@ -203,7 +203,7 @@

Library Stdlib.Reals.Rbasic_fun

-

Rabsolu

+

Rabsolu

diff --git a/master/stdlib/Stdlib.Reals.Rdefinitions.html b/master/stdlib/Stdlib.Reals.Rdefinitions.html index 0bb0ba43ef..5cb4d86db2 100644 --- a/master/stdlib/Stdlib.Reals.Rdefinitions.html +++ b/master/stdlib/Stdlib.Reals.Rdefinitions.html @@ -178,7 +178,7 @@

Library Stdlib.Reals.Rdefinitions

-

Injection from Z to R

+

Injection from Z to R

@@ -266,7 +266,7 @@

Library Stdlib.Reals.Rdefinitions

-

Number notation for constants

+

Number notation for constants

diff --git a/master/stdlib/Stdlib.Reals.Rfunctions.html b/master/stdlib/Stdlib.Reals.Rfunctions.html index c0d1d0a5d2..ad67ac74fa 100644 --- a/master/stdlib/Stdlib.Reals.Rfunctions.html +++ b/master/stdlib/Stdlib.Reals.Rfunctions.html @@ -74,7 +74,7 @@

Library Stdlib.Reals.Rfunctions

-

Lemmas about factorial

+

Lemmas about factorial

@@ -91,7 +91,7 @@

Library Stdlib.Reals.Rfunctions

-

Power

+

Power

@@ -230,7 +230,7 @@

Library Stdlib.Reals.Rfunctions

-

PowerRZ

+

PowerRZ

@@ -379,7 +379,7 @@

Library Stdlib.Reals.Rfunctions

-

Sum of n first naturals

+

Sum of n first naturals

@@ -403,7 +403,7 @@

Library Stdlib.Reals.Rfunctions

-

Sum

+

Sum

@@ -431,7 +431,7 @@

Library Stdlib.Reals.Rfunctions

-

Distance in R

+

Distance in R

@@ -477,7 +477,7 @@

Library Stdlib.Reals.Rfunctions

-

Infinite Sum

+

Infinite Sum

diff --git a/master/stdlib/Stdlib.Reals.Rgeom.html b/master/stdlib/Stdlib.Reals.Rgeom.html index b30a669f7c..a1c396a1a6 100644 --- a/master/stdlib/Stdlib.Reals.Rgeom.html +++ b/master/stdlib/Stdlib.Reals.Rgeom.html @@ -57,7 +57,7 @@

Library Stdlib.Reals.Rgeom

-

Distance

+

Distance

@@ -91,7 +91,7 @@

Library Stdlib.Reals.Rgeom

-

Translation

+

Translation

@@ -113,7 +113,7 @@

Library Stdlib.Reals.Rgeom

-

Rotation

+

Rotation

@@ -147,7 +147,7 @@

Library Stdlib.Reals.Rgeom

-

Similarity

+

Similarity

diff --git a/master/stdlib/Stdlib.Reals.RiemannInt_SF.html b/master/stdlib/Stdlib.Reals.RiemannInt_SF.html index 3b5fed5c43..632d78de0b 100644 --- a/master/stdlib/Stdlib.Reals.RiemannInt_SF.html +++ b/master/stdlib/Stdlib.Reals.RiemannInt_SF.html @@ -62,7 +62,7 @@

Library Stdlib.Reals.RiemannInt_SF

-

Each bounded subset of N has a maximal element

+

Each bounded subset of N has a maximal element

@@ -84,7 +84,7 @@

Library Stdlib.Reals.RiemannInt_SF

-

Step functions

+

Step functions

@@ -124,7 +124,7 @@

Library Stdlib.Reals.RiemannInt_SF

-

Class of step functions

+

Class of step functions

@@ -156,7 +156,7 @@

Library Stdlib.Reals.RiemannInt_SF

-

Integral of step functions

+

Integral of step functions

@@ -170,7 +170,7 @@

Library Stdlib.Reals.RiemannInt_SF

-

Properties of step functions

+

Properties of step functions

diff --git a/master/stdlib/Stdlib.Reals.Rlimit.html b/master/stdlib/Stdlib.Reals.Rlimit.html index c4e2b98433..79d2560141 100644 --- a/master/stdlib/Stdlib.Reals.Rlimit.html +++ b/master/stdlib/Stdlib.Reals.Rlimit.html @@ -63,7 +63,7 @@

Library Stdlib.Reals.Rlimit

-

Calculus

+

Calculus

@@ -101,7 +101,7 @@

Library Stdlib.Reals.Rlimit

-

Metric space

+

Metric space

@@ -120,7 +120,7 @@

Library Stdlib.Reals.Rlimit

-

Limit in Metric space

+

Limit in Metric space

@@ -139,7 +139,7 @@

Library Stdlib.Reals.Rlimit

-

R is a metric space

+

R is a metric space

@@ -155,7 +155,7 @@

Library Stdlib.Reals.Rlimit

-

Limit 1 arg

+

Limit 1 arg

diff --git a/master/stdlib/Stdlib.Reals.Rlogic.html b/master/stdlib/Stdlib.Reals.Rlogic.html index a67e96f95b..7212ecf595 100644 --- a/master/stdlib/Stdlib.Reals.Rlogic.html +++ b/master/stdlib/Stdlib.Reals.Rlogic.html @@ -75,7 +75,7 @@

Library Stdlib.Reals.Rlogic

-

Decidability of arithmetical statements

+

Decidability of arithmetical statements

@@ -101,7 +101,7 @@

Library Stdlib.Reals.Rlogic

-

Derivability of the Archimedean axiom

+

Derivability of the Archimedean axiom

@@ -121,7 +121,7 @@

Library Stdlib.Reals.Rlogic

-

Decidability of negated formulas

+

Decidability of negated formulas

diff --git a/master/stdlib/Stdlib.Reals.Rminmax.html b/master/stdlib/Stdlib.Reals.Rminmax.html index b62fd713d6..09fcfc2fbd 100644 --- a/master/stdlib/Stdlib.Reals.Rminmax.html +++ b/master/stdlib/Stdlib.Reals.Rminmax.html @@ -55,7 +55,7 @@

Library Stdlib.Reals.Rminmax

-

Maximum and Minimum of two real numbers

+

Maximum and Minimum of two real numbers

@@ -112,7 +112,7 @@

Library Stdlib.Reals.Rminmax

-

Properties specific to the R domain

+

Properties specific to the R domain

diff --git a/master/stdlib/Stdlib.Reals.Rpower.html b/master/stdlib/Stdlib.Reals.Rpower.html index d5d323711e..a67fde76f8 100644 --- a/master/stdlib/Stdlib.Reals.Rpower.html +++ b/master/stdlib/Stdlib.Reals.Rpower.html @@ -76,7 +76,7 @@

Library Stdlib.Reals.Rpower

-

Properties of Exp

+

Properties of Exp

@@ -129,7 +129,7 @@

Library Stdlib.Reals.Rpower

-

Properties of Ln

+

Properties of Ln

@@ -169,7 +169,7 @@

Library Stdlib.Reals.Rpower

-

Definition of Rpower

+

Definition of Rpower

@@ -181,7 +181,7 @@

Library Stdlib.Reals.Rpower

-

Properties of Rpower

+

Properties of Rpower

@@ -248,7 +248,7 @@

Library Stdlib.Reals.Rpower

-

Differentiability of Ln and Rpower

+

Differentiability of Ln and Rpower

diff --git a/master/stdlib/Stdlib.Reals.Rseries.html b/master/stdlib/Stdlib.Reals.Rseries.html index 3438f16657..b85e86f9a2 100644 --- a/master/stdlib/Stdlib.Reals.Rseries.html +++ b/master/stdlib/Stdlib.Reals.Rseries.html @@ -58,7 +58,7 @@

Library Stdlib.Reals.Rseries

-

Definition of sequence and properties

+

Definition of sequence and properties

@@ -130,7 +130,7 @@

Library Stdlib.Reals.Rseries

-

Definition of Power Series and properties

+

Definition of Power Series and properties

diff --git a/master/stdlib/Stdlib.Reals.Rtopology.html b/master/stdlib/Stdlib.Reals.Rtopology.html index 35587b5aee..c1ca8c173c 100644 --- a/master/stdlib/Stdlib.Reals.Rtopology.html +++ b/master/stdlib/Stdlib.Reals.Rtopology.html @@ -59,7 +59,7 @@

Library Stdlib.Reals.Rtopology

-

General definitions and propositions

+

General definitions and propositions

@@ -307,7 +307,7 @@

Library Stdlib.Reals.Rtopology

-

Proof of Bolzano-Weierstrass theorem

+

Proof of Bolzano-Weierstrass theorem

@@ -380,7 +380,7 @@

Library Stdlib.Reals.Rtopology

-

Proof of Heine's theorem

+

Proof of Heine's theorem

diff --git a/master/stdlib/Stdlib.Reals.Rtrigo1.html b/master/stdlib/Stdlib.Reals.Rtrigo1.html index cc6d662efc..93f3b42ca9 100644 --- a/master/stdlib/Stdlib.Reals.Rtrigo1.html +++ b/master/stdlib/Stdlib.Reals.Rtrigo1.html @@ -164,7 +164,7 @@

Library Stdlib.Reals.Rtrigo1

-

Some properties of cos, sin and tan

+

Some properties of cos, sin and tan

@@ -258,7 +258,7 @@

Library Stdlib.Reals.Rtrigo1

-

Using series definitions of cos and sin

+

Using series definitions of cos and sin

@@ -292,7 +292,7 @@

Library Stdlib.Reals.Rtrigo1

-

Increasing and decreasing of cos and sin

+

Increasing and decreasing of cos and sin

diff --git a/master/stdlib/Stdlib.Reals.Rtrigo_def.html b/master/stdlib/Stdlib.Reals.Rtrigo_def.html index c4bfa207ba..efb7776fc2 100644 --- a/master/stdlib/Stdlib.Reals.Rtrigo_def.html +++ b/master/stdlib/Stdlib.Reals.Rtrigo_def.html @@ -54,7 +54,7 @@

Library Stdlib.Reals.Rtrigo_def

-

Definition of exponential

+

Definition of exponential

@@ -80,7 +80,7 @@

Library Stdlib.Reals.Rtrigo_def

-

Definition of hyperbolic functions

+

Definition of hyperbolic functions

@@ -154,7 +154,7 @@

Library Stdlib.Reals.Rtrigo_def

-

Properties

+

Properties

diff --git a/master/stdlib/Stdlib.Reals.Rtrigo_facts.html b/master/stdlib/Stdlib.Reals.Rtrigo_facts.html index 65d2c6da01..03ab5ba562 100644 --- a/master/stdlib/Stdlib.Reals.Rtrigo_facts.html +++ b/master/stdlib/Stdlib.Reals.Rtrigo_facts.html @@ -61,7 +61,7 @@

Library Stdlib.Reals.Rtrigo_facts

-

Bounds of expressions with trigonometric functions

+

Bounds of expressions with trigonometric functions

@@ -78,11 +78,11 @@

Library Stdlib.Reals.Rtrigo_facts

-

Express trigonometric functions with each other

+

Express trigonometric functions with each other

-

Express sin and cos with each other

+

Express sin and cos with each other

@@ -115,7 +115,7 @@

Library Stdlib.Reals.Rtrigo_facts

-

Express tan with sin and cos

+

Express tan with sin and cos

@@ -148,7 +148,7 @@

Library Stdlib.Reals.Rtrigo_facts

-

Express sin and cos with tan

+

Express sin and cos with tan

@@ -165,7 +165,7 @@

Library Stdlib.Reals.Rtrigo_facts

-

Additional shift lemmas for sin, cos, tan

+

Additional shift lemmas for sin, cos, tan

diff --git a/master/stdlib/Stdlib.Relations.Operators_Properties.html b/master/stdlib/Stdlib.Relations.Operators_Properties.html index f6f999797b..acb3c15a89 100644 --- a/master/stdlib/Stdlib.Relations.Operators_Properties.html +++ b/master/stdlib/Stdlib.Relations.Operators_Properties.html @@ -49,8 +49,8 @@

Library Stdlib.Relations.Operators_Properties

-

Some properties of the operators on relations

-

Initial version by Bruno Barras

+

Some properties of the operators on relations

+

Initial version by Bruno Barras

@@ -185,12 +185,12 @@

Library Stdlib.Relations.Operators_Properties

-

Equivalences between the different definition of the reflexive,

+

Equivalences between the different definition of the reflexive,

symmetric, transitive closures
-

Contributed by P. Castéran

+

Contributed by P. Castéran

diff --git a/master/stdlib/Stdlib.Relations.Relation_Operators.html b/master/stdlib/Stdlib.Relations.Relation_Operators.html index dd94f1d160..3b1d428dfb 100644 --- a/master/stdlib/Stdlib.Relations.Relation_Operators.html +++ b/master/stdlib/Stdlib.Relations.Relation_Operators.html @@ -49,14 +49,14 @@

Library Stdlib.Relations.Relation_Operators

-

Some operators on relations

-

Initial authors: Bruno Barras, Cristina Cornes

-

-

Some of the initial definitions were taken from :

-

Constructing Recursion Operators in Type Theory

-

L. Paulson JSC (1986) 2, 325-355

-

-

Further extensions by Pierre Castéran

+

Some operators on relations

+

Initial authors: Bruno Barras, Cristina Cornes

+

+

Some of the initial definitions were taken from :

+

Constructing Recursion Operators in Type Theory

+

L. Paulson JSC (1986) 2, 325-355

+

+

Further extensions by Pierre Castéran

@@ -68,7 +68,7 @@

Library Stdlib.Relations.Relation_Operators

-

Transitive closure

+

Transitive closure

@@ -124,7 +124,7 @@

Library Stdlib.Relations.Relation_Operators

-

Reflexive closure

+

Reflexive closure

@@ -154,7 +154,7 @@

Library Stdlib.Relations.Relation_Operators

-

Reflexive-transitive closure

+

Reflexive-transitive closure

@@ -214,7 +214,7 @@

Library Stdlib.Relations.Relation_Operators

-

Reflexive-symmetric-transitive closure

+

Reflexive-symmetric-transitive closure

@@ -276,7 +276,7 @@

Library Stdlib.Relations.Relation_Operators

-

Converse of a relation

+

Converse of a relation

@@ -294,7 +294,7 @@

Library Stdlib.Relations.Relation_Operators

-

Union of relations

+

Union of relations

@@ -312,7 +312,7 @@

Library Stdlib.Relations.Relation_Operators

-

Disjoint union of relations

+

Disjoint union of relations

@@ -336,7 +336,7 @@

Library Stdlib.Relations.Relation_Operators

-

Lexicographic order on dependent pairs

+

Lexicographic order on dependent pairs

@@ -369,7 +369,7 @@

Library Stdlib.Relations.Relation_Operators

-

Lexicographic order on pairs

+

Lexicographic order on pairs

@@ -404,7 +404,7 @@

Library Stdlib.Relations.Relation_Operators

-

Product of relations

+

Product of relations

@@ -430,7 +430,7 @@

Library Stdlib.Relations.Relation_Operators

-

Multiset of two relations

+

Multiset of two relations

diff --git a/master/stdlib/Stdlib.Sorting.CPermutation.html b/master/stdlib/Stdlib.Sorting.CPermutation.html index b5b1a7c57a..9b23ff17d0 100644 --- a/master/stdlib/Stdlib.Sorting.CPermutation.html +++ b/master/stdlib/Stdlib.Sorting.CPermutation.html @@ -49,7 +49,7 @@

Library Stdlib.Sorting.CPermutation

-

Circular Shifts (aka Cyclic Permutations)

+

Circular Shifts (aka Cyclic Permutations)

diff --git a/master/stdlib/Stdlib.Sorting.Heap.html b/master/stdlib/Stdlib.Sorting.Heap.html index c38c2d53d2..3c1c9581d4 100644 --- a/master/stdlib/Stdlib.Sorting.Heap.html +++ b/master/stdlib/Stdlib.Sorting.Heap.html @@ -74,11 +74,11 @@

Library Stdlib.Sorting.Heap

-

Trees and heap trees

+

Trees and heap trees

-

Definition of trees over an ordered set

+

Definition of trees over an ordered set

@@ -143,7 +143,7 @@

Library Stdlib.Sorting.Heap

-

The heap property

+

The heap property

@@ -195,7 +195,7 @@

Library Stdlib.Sorting.Heap

-

Merging two sorted lists

+

Merging two sorted lists

@@ -227,7 +227,7 @@

Library Stdlib.Sorting.Heap

-

From trees to multisets

+

From trees to multisets

@@ -263,11 +263,11 @@

Library Stdlib.Sorting.Heap

-

From lists to sorted lists

+

From lists to sorted lists

-

Specification of heap insertion

+

Specification of heap insertion

@@ -289,7 +289,7 @@

Library Stdlib.Sorting.Heap

-

Building a heap from a list

+

Building a heap from a list

@@ -309,7 +309,7 @@

Library Stdlib.Sorting.Heap

-

Building the sorted list

+

Building the sorted list

@@ -330,7 +330,7 @@

Library Stdlib.Sorting.Heap

-

Specification of treesort

+

Specification of treesort

diff --git a/master/stdlib/Stdlib.Sorting.PermutSetoid.html b/master/stdlib/Stdlib.Sorting.PermutSetoid.html index 6c305bad78..ee6af92e4d 100644 --- a/master/stdlib/Stdlib.Sorting.PermutSetoid.html +++ b/master/stdlib/Stdlib.Sorting.PermutSetoid.html @@ -89,7 +89,7 @@

Library Stdlib.Sorting.PermutSetoid

-

From lists to multisets

+

From lists to multisets

@@ -128,7 +128,7 @@

Library Stdlib.Sorting.PermutSetoid

-

permutation: definition and basic properties

+

permutation: definition and basic properties

@@ -202,7 +202,7 @@

Library Stdlib.Sorting.PermutSetoid

-

Some inversion results.

+

Some inversion results.

diff --git a/master/stdlib/Stdlib.Sorting.Permutation.html b/master/stdlib/Stdlib.Sorting.Permutation.html index 4a3abd133d..f8ff8da32a 100644 --- a/master/stdlib/Stdlib.Sorting.Permutation.html +++ b/master/stdlib/Stdlib.Sorting.Permutation.html @@ -49,7 +49,7 @@

Library Stdlib.Sorting.Permutation

-

List permutations as a composition of adjacent transpositions

+

List permutations as a composition of adjacent transpositions

diff --git a/master/stdlib/Stdlib.Strings.Ascii.html b/master/stdlib/Stdlib.Strings.Ascii.html index ffec23609c..064118d0f5 100644 --- a/master/stdlib/Stdlib.Strings.Ascii.html +++ b/master/stdlib/Stdlib.Strings.Ascii.html @@ -62,7 +62,7 @@

Library Stdlib.Strings.Ascii

-

Definition of ascii characters

+

Definition of ascii characters

@@ -142,7 +142,7 @@

Library Stdlib.Strings.Ascii

-

Conversion between natural numbers modulo 256 and ascii characters

+

Conversion between natural numbers modulo 256 and ascii characters

@@ -284,7 +284,7 @@

Library Stdlib.Strings.Ascii

-

Concrete syntax

+

Concrete syntax

diff --git a/master/stdlib/Stdlib.Strings.PString.html b/master/stdlib/Stdlib.Strings.PString.html index 6e9c8541cb..c9c3b760c9 100644 --- a/master/stdlib/Stdlib.Strings.PString.html +++ b/master/stdlib/Stdlib.Strings.PString.html @@ -128,7 +128,7 @@

Library Stdlib.Strings.PString

-

Properties of string length

+

Properties of string length

@@ -169,7 +169,7 @@

Library Stdlib.Strings.PString

-

Properties of string get

+

Properties of string get

@@ -212,7 +212,7 @@

Library Stdlib.Strings.PString

-

Properties of string comparison

+

Properties of string comparison

@@ -293,7 +293,7 @@

Library Stdlib.Strings.PString

-

Properties of make

+

Properties of make

@@ -305,7 +305,7 @@

Library Stdlib.Strings.PString

-

Properties of cat

+

Properties of cat

@@ -327,7 +327,7 @@

Library Stdlib.Strings.PString

-

Properties of sub

+

Properties of sub

@@ -375,7 +375,7 @@

Library Stdlib.Strings.PString

-

Ordered type

+

Ordered type

diff --git a/master/stdlib/Stdlib.Strings.PrimStringAxioms.html b/master/stdlib/Stdlib.Strings.PrimStringAxioms.html index a93656694d..32ff049110 100644 --- a/master/stdlib/Stdlib.Strings.PrimStringAxioms.html +++ b/master/stdlib/Stdlib.Strings.PrimStringAxioms.html @@ -56,7 +56,7 @@

Library Stdlib.Strings.PrimStringAxioms

-

Conversion to / from lists

+

Conversion to / from lists

@@ -91,7 +91,7 @@

Library Stdlib.Strings.PrimStringAxioms

-

Axioms relating string operations with list operations

+

Axioms relating string operations with list operations

diff --git a/master/stdlib/Stdlib.Strings.String.html b/master/stdlib/Stdlib.Strings.String.html index 359f7ddd94..d15ede72a4 100644 --- a/master/stdlib/Stdlib.Strings.String.html +++ b/master/stdlib/Stdlib.Strings.String.html @@ -65,7 +65,7 @@

Library Stdlib.Strings.String

-

Definition of strings

+

Definition of strings

@@ -136,7 +136,7 @@

Library Stdlib.Strings.String

-

Compare strings lexicographically

+

Compare strings lexicographically

@@ -186,7 +186,7 @@

Library Stdlib.Strings.String

-

Concatenation of strings

+

Concatenation of strings

@@ -277,7 +277,7 @@

Library Stdlib.Strings.String

-

Substrings

+

Substrings

@@ -326,7 +326,7 @@

Library Stdlib.Strings.String

-

Concatenating lists of strings

+

Concatenating lists of strings

@@ -347,7 +347,7 @@

Library Stdlib.Strings.String

-

Test functions

+

Test functions

@@ -499,7 +499,7 @@

Library Stdlib.Strings.String

-

Conversion to/from list ascii and list byte

+

Conversion to/from list ascii and list byte

@@ -542,7 +542,7 @@

Library Stdlib.Strings.String

-

Concrete syntax

+

Concrete syntax

diff --git a/master/stdlib/Stdlib.Structures.DecidableType.html b/master/stdlib/Stdlib.Structures.DecidableType.html index f6e569e3d1..ffb1a9ca0f 100644 --- a/master/stdlib/Stdlib.Structures.DecidableType.html +++ b/master/stdlib/Stdlib.Structures.DecidableType.html @@ -60,7 +60,7 @@

Library Stdlib.Structures.DecidableType

FSets and FMap. Please use Structures/Equalities.v directly now.
-

Types with Equalities, and nothing more (for subtyping purpose)

+

Types with Equalities, and nothing more (for subtyping purpose)

@@ -72,7 +72,7 @@

Library Stdlib.Structures.DecidableType

-

Types with decidable Equalities (but no ordering)

+

Types with decidable Equalities (but no ordering)

@@ -84,7 +84,7 @@

Library Stdlib.Structures.DecidableType

-

Additional notions about keys and datas used in FMap

+

Additional notions about keys and datas used in FMap

diff --git a/master/stdlib/Stdlib.Structures.DecidableTypeEx.html b/master/stdlib/Stdlib.Structures.DecidableTypeEx.html index 6c54c6a9f9..66742a0683 100644 --- a/master/stdlib/Stdlib.Structures.DecidableTypeEx.html +++ b/master/stdlib/Stdlib.Structures.DecidableTypeEx.html @@ -57,7 +57,7 @@

Library Stdlib.Structures.DecidableTypeEx

FSets and FMap. Please use Structures/Equalities.v directly now.
-

Examples of Decidable Type structures.

+

Examples of Decidable Type structures.

diff --git a/master/stdlib/Stdlib.Structures.Equalities.html b/master/stdlib/Stdlib.Structures.Equalities.html index cba72ec21e..9ec01ca262 100644 --- a/master/stdlib/Stdlib.Structures.Equalities.html +++ b/master/stdlib/Stdlib.Structures.Equalities.html @@ -69,7 +69,7 @@

Library Stdlib.Structures.Equalities

-

Structure with just a base type t

+

Structure with just a base type t

@@ -83,7 +83,7 @@

Library Stdlib.Structures.Equalities

-

Structure with an equality relation eq

+

Structure with an equality relation eq

@@ -109,7 +109,7 @@

Library Stdlib.Structures.Equalities

-

Specification of the equality via the Equivalence type class

+

Specification of the equality via the Equivalence type class

@@ -124,7 +124,7 @@

Library Stdlib.Structures.Equalities

-

Earlier specification of equality by three separate lemmas.

+

Earlier specification of equality by three separate lemmas.

@@ -144,7 +144,7 @@

Library Stdlib.Structures.Equalities

-

Types with decidable equality

+

Types with decidable equality

@@ -158,7 +158,7 @@

Library Stdlib.Structures.Equalities

-

Boolean Equality

+

Boolean Equality

@@ -253,7 +253,7 @@

Library Stdlib.Structures.Equalities

-

Compatibility wrapper from/to the old version of

+

Compatibility wrapper from/to the old version of

EqualityType and DecidableType
@@ -292,7 +292,7 @@

Library Stdlib.Structures.Equalities

-

Having eq_dec is equivalent to having eqb and its spec.

+

Having eq_dec is equivalent to having eqb and its spec.

@@ -390,7 +390,7 @@

Library Stdlib.Structures.Equalities

-

UsualDecidableType

+

UsualDecidableType

diff --git a/master/stdlib/Stdlib.Structures.EqualitiesFacts.html b/master/stdlib/Stdlib.Structures.EqualitiesFacts.html index 2d59142007..5a1df74c66 100644 --- a/master/stdlib/Stdlib.Structures.EqualitiesFacts.html +++ b/master/stdlib/Stdlib.Structures.EqualitiesFacts.html @@ -55,7 +55,7 @@

Library Stdlib.Structures.EqualitiesFacts

-

Keys and datas used in the future MMaps

+

Keys and datas used in the future MMaps

@@ -227,7 +227,7 @@

Library Stdlib.Structures.EqualitiesFacts

-

PairDecidableType

+

PairDecidableType

diff --git a/master/stdlib/Stdlib.Structures.GenericMinMax.html b/master/stdlib/Stdlib.Structures.GenericMinMax.html index c4c5ebcd56..9ea47a8920 100644 --- a/master/stdlib/Stdlib.Structures.GenericMinMax.html +++ b/master/stdlib/Stdlib.Structures.GenericMinMax.html @@ -52,11 +52,11 @@

Library Stdlib.Structures.GenericMinMax

-

A Generic construction of min and max

+

A Generic construction of min and max

-

First, an interface for types with max and/or min

+

First, an interface for types with max and/or min

@@ -82,7 +82,7 @@

Library Stdlib.Structures.GenericMinMax

-

Any OrderedTypeFull can be equipped by max and min

+

Any OrderedTypeFull can be equipped by max and min

based on the compare function.
@@ -123,7 +123,7 @@

Library Stdlib.Structures.GenericMinMax

-

Consequences of the minimalist interface: facts about max and min.

+

Consequences of the minimalist interface: facts about max and min.

@@ -201,7 +201,7 @@

Library Stdlib.Structures.GenericMinMax

-

Semi-lattice algebraic properties of max

+

Semi-lattice algebraic properties of max

@@ -228,7 +228,7 @@

Library Stdlib.Structures.GenericMinMax

-

Least-upper bound properties of max

+

Least-upper bound properties of max

@@ -387,7 +387,7 @@

Library Stdlib.Structures.GenericMinMax

-

Combined properties of min and max

+

Combined properties of min and max

@@ -469,7 +469,7 @@

Library Stdlib.Structures.GenericMinMax

-

Properties requiring a decidable order

+

Properties requiring a decidable order

@@ -549,7 +549,7 @@

Library Stdlib.Structures.GenericMinMax

-

When the equality is Leibniz, we can skip a few Proper precondition.

+

When the equality is Leibniz, we can skip a few Proper precondition.

diff --git a/master/stdlib/Stdlib.Structures.OrderedType.html b/master/stdlib/Stdlib.Structures.OrderedType.html index 2c3f0ed6bb..b7643e335a 100644 --- a/master/stdlib/Stdlib.Structures.OrderedType.html +++ b/master/stdlib/Stdlib.Structures.OrderedType.html @@ -57,7 +57,7 @@

Library Stdlib.Structures.OrderedType

FSets and FMap. Please use Structures/Orders.v directly now.
-

Ordered types

+

Ordered types

@@ -138,7 +138,7 @@

Library Stdlib.Structures.OrderedType

-

Ordered types properties

+

Ordered types properties

diff --git a/master/stdlib/Stdlib.Structures.OrderedTypeAlt.html b/master/stdlib/Stdlib.Structures.OrderedTypeAlt.html index 0513d21122..4ae99807c7 100644 --- a/master/stdlib/Stdlib.Structures.OrderedTypeAlt.html +++ b/master/stdlib/Stdlib.Structures.OrderedTypeAlt.html @@ -50,7 +50,7 @@

Library Stdlib.Structures.OrderedTypeAlt

-

An alternative (but equivalent) presentation for an Ordered Type

+

An alternative (but equivalent) presentation for an Ordered Type

inferface.
diff --git a/master/stdlib/Stdlib.Structures.OrderedTypeEx.html b/master/stdlib/Stdlib.Structures.OrderedTypeEx.html index 1aad3b13f8..4bf74b5fa5 100644 --- a/master/stdlib/Stdlib.Structures.OrderedTypeEx.html +++ b/master/stdlib/Stdlib.Structures.OrderedTypeEx.html @@ -56,7 +56,7 @@

Library Stdlib.Structures.OrderedTypeEx

-

Examples of Ordered Type structures.

+

Examples of Ordered Type structures.

diff --git a/master/stdlib/Stdlib.Structures.Orders.html b/master/stdlib/Stdlib.Structures.Orders.html index 513f41977f..811b159461 100644 --- a/master/stdlib/Stdlib.Structures.Orders.html +++ b/master/stdlib/Stdlib.Structures.Orders.html @@ -53,7 +53,7 @@

Library Stdlib.Structures.Orders

-

Ordered types

+

Ordered types

@@ -188,7 +188,7 @@

Library Stdlib.Structures.Orders

DecidableType.
-

Versions with eq being the usual Leibniz equality of Coq

+

Versions with eq being the usual Leibniz equality of Coq

@@ -220,7 +220,7 @@

Library Stdlib.Structures.Orders

-

Purely logical versions

+

Purely logical versions

@@ -243,7 +243,7 @@

Library Stdlib.Structures.Orders

-

Conversions

+

Conversions

@@ -304,7 +304,7 @@

Library Stdlib.Structures.Orders

-

Versions with boolean comparisons

+

Versions with boolean comparisons

@@ -406,7 +406,7 @@

Library Stdlib.Structures.Orders

-

From OrderedTypeFull to TotalTransitiveLeBool

+

From OrderedTypeFull to TotalTransitiveLeBool

@@ -437,7 +437,7 @@

Library Stdlib.Structures.Orders

-

From TotalTransitiveLeBool to OrderedTypeFull

+

From TotalTransitiveLeBool to OrderedTypeFull

diff --git a/master/stdlib/Stdlib.Structures.OrdersAlt.html b/master/stdlib/Stdlib.Structures.OrdersAlt.html index 932ac2aa69..b5e02aad68 100644 --- a/master/stdlib/Stdlib.Structures.OrdersAlt.html +++ b/master/stdlib/Stdlib.Structures.OrdersAlt.html @@ -55,12 +55,12 @@

Library Stdlib.Structures.OrdersAlt

-

Some alternative (but equivalent) presentations for an Ordered Type

+

Some alternative (but equivalent) presentations for an Ordered Type

inferface.
-

The original interface

+

The original interface

@@ -72,7 +72,7 @@

Library Stdlib.Structures.OrdersAlt

-

An interface based on compare

+

An interface based on compare

@@ -102,7 +102,7 @@

Library Stdlib.Structures.OrdersAlt

-

From OrderedTypeOrig to OrderedType.

+

From OrderedTypeOrig to OrderedType.

@@ -141,7 +141,7 @@

Library Stdlib.Structures.OrdersAlt

-

From OrderedType to OrderedTypeOrig.

+

From OrderedType to OrderedTypeOrig.

@@ -170,7 +170,7 @@

Library Stdlib.Structures.OrdersAlt

-

From OrderedTypeAlt to OrderedType.

+

From OrderedTypeAlt to OrderedType.

diff --git a/master/stdlib/Stdlib.Structures.OrdersEx.html b/master/stdlib/Stdlib.Structures.OrdersEx.html index 97a5414258..e4e83f8792 100644 --- a/master/stdlib/Stdlib.Structures.OrdersEx.html +++ b/master/stdlib/Stdlib.Structures.OrdersEx.html @@ -56,7 +56,7 @@

Library Stdlib.Structures.OrdersEx

-

Examples of Ordered Type structures.

+

Examples of Ordered Type structures.

diff --git a/master/stdlib/Stdlib.Structures.OrdersFacts.html b/master/stdlib/Stdlib.Structures.OrdersFacts.html index a4f6dba472..12e77cb7a0 100644 --- a/master/stdlib/Stdlib.Structures.OrdersFacts.html +++ b/master/stdlib/Stdlib.Structures.OrdersFacts.html @@ -56,7 +56,7 @@

Library Stdlib.Structures.OrdersFacts

-

Properties of compare

+

Properties of compare

@@ -105,7 +105,7 @@

Library Stdlib.Structures.OrdersFacts

-

Properties of OrderedTypeFull

+

Properties of OrderedTypeFull

@@ -165,7 +165,7 @@

Library Stdlib.Structures.OrdersFacts

-

Properties of OrderedType

+

Properties of OrderedType

@@ -260,7 +260,7 @@

Library Stdlib.Structures.OrdersFacts

-

Tests of the order tactic

+

Tests of the order tactic

@@ -298,7 +298,7 @@

Library Stdlib.Structures.OrdersFacts

-

Reversed OrderedTypeFull.

+

Reversed OrderedTypeFull.

@@ -349,7 +349,7 @@

Library Stdlib.Structures.OrdersFacts

-

Order relations derived from a compare function.

+

Order relations derived from a compare function.

diff --git a/master/stdlib/Stdlib.Structures.OrdersLists.html b/master/stdlib/Stdlib.Structures.OrdersLists.html index 04ebb264ea..2dba225a5e 100644 --- a/master/stdlib/Stdlib.Structures.OrdersLists.html +++ b/master/stdlib/Stdlib.Structures.OrdersLists.html @@ -55,7 +55,7 @@

Library Stdlib.Structures.OrdersLists

-

Specialization of results about lists modulo.

+

Specialization of results about lists modulo.

@@ -110,7 +110,7 @@

Library Stdlib.Structures.OrdersLists

-

Results about keys and data as manipulated in the future MMaps.

+

Results about keys and data as manipulated in the future MMaps.

diff --git a/master/stdlib/Stdlib.Structures.OrdersTac.html b/master/stdlib/Stdlib.Structures.OrdersTac.html index 9a02089023..10f698a0e3 100644 --- a/master/stdlib/Stdlib.Structures.OrdersTac.html +++ b/master/stdlib/Stdlib.Structures.OrdersTac.html @@ -53,7 +53,7 @@

Library Stdlib.Structures.OrdersTac

-

The order tactic

+

The order tactic

@@ -92,7 +92,7 @@

Library Stdlib.Structures.OrdersTac

-

The tactic requirements : a total order

+

The tactic requirements : a total order

@@ -128,7 +128,7 @@

Library Stdlib.Structures.OrdersTac

-

Properties that will be used by the order tactic

+

Properties that will be used by the order tactic

@@ -238,7 +238,7 @@

Library Stdlib.Structures.OrdersTac

-

MakeOrderTac : The functor providing the order tactic.

+

MakeOrderTac : The functor providing the order tactic.

diff --git a/master/stdlib/Stdlib.Vectors.VectorDef.html b/master/stdlib/Stdlib.Vectors.VectorDef.html index 6c8bf4a1c9..70200685b5 100644 --- a/master/stdlib/Stdlib.Vectors.VectorDef.html +++ b/master/stdlib/Stdlib.Vectors.VectorDef.html @@ -437,7 +437,7 @@

Library Stdlib.Vectors.VectorDef

-

Here are special non dependent useful instantiation of induction schemes

+

Here are special non dependent useful instantiation of induction schemes

@@ -564,7 +564,7 @@

Library Stdlib.Vectors.VectorDef

-

vector <=> list functions

+

vector <=> list functions

diff --git a/master/stdlib/Stdlib.Vectors.VectorSpec.html b/master/stdlib/Stdlib.Vectors.VectorSpec.html index d0dd0e9475..a8050c7f6a 100644 --- a/master/stdlib/Stdlib.Vectors.VectorSpec.html +++ b/master/stdlib/Stdlib.Vectors.VectorSpec.html @@ -95,7 +95,7 @@

Library Stdlib.Vectors.VectorSpec

is true for the one that use lt
-

Properties of nth and nth_order

+

Properties of nth and nth_order

@@ -136,7 +136,7 @@

Library Stdlib.Vectors.VectorSpec

-

Properties of replace

+

Properties of replace

@@ -182,7 +182,7 @@

Library Stdlib.Vectors.VectorSpec

-

Properties of const

+

Properties of const

@@ -197,7 +197,7 @@

Library Stdlib.Vectors.VectorSpec

-

Properties of map

+

Properties of map

@@ -238,7 +238,7 @@

Library Stdlib.Vectors.VectorSpec

-

Properties of fold_left

+

Properties of fold_left

@@ -252,7 +252,7 @@

Library Stdlib.Vectors.VectorSpec

-

Properties of take

+

Properties of take

@@ -274,7 +274,7 @@

Library Stdlib.Vectors.VectorSpec

-

Properties of uncons and splitat

+

Properties of uncons and splitat

@@ -305,7 +305,7 @@

Library Stdlib.Vectors.VectorSpec

-

Properties of In

+

Properties of In

@@ -318,7 +318,7 @@

Library Stdlib.Vectors.VectorSpec

-

Properties of Forall and Forall2

+

Properties of Forall and Forall2

@@ -372,7 +372,7 @@

Library Stdlib.Vectors.VectorSpec

-

Properties of shiftin and shiftrepeat

+

Properties of shiftin and shiftrepeat

@@ -411,7 +411,7 @@

Library Stdlib.Vectors.VectorSpec

-

Properties of rev

+

Properties of rev

@@ -449,7 +449,7 @@

Library Stdlib.Vectors.VectorSpec

-

Properties of to_list

+

Properties of to_list

diff --git a/master/stdlib/Stdlib.ZArith.BinInt.html b/master/stdlib/Stdlib.ZArith.BinInt.html index 8903302047..3339a7ab54 100644 --- a/master/stdlib/Stdlib.ZArith.BinInt.html +++ b/master/stdlib/Stdlib.ZArith.BinInt.html @@ -55,7 +55,7 @@

Library Stdlib.ZArith.BinInt

-

Binary Integers

+

Binary Integers

@@ -90,7 +90,7 @@

Library Stdlib.ZArith.BinInt

-

Definitions of operations, now in a separate file

+

Definitions of operations, now in a separate file

@@ -122,7 +122,7 @@

Library Stdlib.ZArith.BinInt

-

Logic Predicates

+

Logic Predicates

@@ -172,7 +172,7 @@

Library Stdlib.ZArith.BinInt

-

Decidability of equality.

+

Decidability of equality.

@@ -184,7 +184,7 @@

Library Stdlib.ZArith.BinInt

-

Proofs of morphisms, obvious since eq is Leibniz

+

Proofs of morphisms, obvious since eq is Leibniz

@@ -209,7 +209,7 @@

Library Stdlib.ZArith.BinInt

-

Properties of pos_sub

+

Properties of pos_sub

@@ -280,7 +280,7 @@

Library Stdlib.ZArith.BinInt

-

Operations and constants

+

Operations and constants

@@ -298,7 +298,7 @@

Library Stdlib.ZArith.BinInt

-

Addition is commutative

+

Addition is commutative

@@ -310,7 +310,7 @@

Library Stdlib.ZArith.BinInt

-

Opposite distributes over addition

+

Opposite distributes over addition

@@ -322,7 +322,7 @@

Library Stdlib.ZArith.BinInt

-

Opposite is injective

+

Opposite is injective

@@ -334,7 +334,7 @@

Library Stdlib.ZArith.BinInt

-

Addition is associative

+

Addition is associative

@@ -356,7 +356,7 @@

Library Stdlib.ZArith.BinInt

-

Opposite is inverse for addition

+

Opposite is inverse for addition

@@ -368,7 +368,7 @@

Library Stdlib.ZArith.BinInt

-

Multiplication and Opposite

+

Multiplication and Opposite

@@ -380,7 +380,7 @@

Library Stdlib.ZArith.BinInt

-

Distributivity of multiplication over addition

+

Distributivity of multiplication over addition

@@ -399,11 +399,11 @@

Library Stdlib.ZArith.BinInt

-

Proofs of specifications

+

Proofs of specifications

-

Specification of constants

+

Specification of constants

@@ -418,7 +418,7 @@

Library Stdlib.ZArith.BinInt

-

Specification of addition

+

Specification of addition

@@ -433,7 +433,7 @@

Library Stdlib.ZArith.BinInt

-

Specification of opposite

+

Specification of opposite

@@ -448,7 +448,7 @@

Library Stdlib.ZArith.BinInt

-

Specification of successor and predecessor

+

Specification of successor and predecessor

@@ -466,7 +466,7 @@

Library Stdlib.ZArith.BinInt

-

Specification of subtraction

+

Specification of subtraction

@@ -481,7 +481,7 @@

Library Stdlib.ZArith.BinInt

-

Specification of multiplication

+

Specification of multiplication

@@ -496,7 +496,7 @@

Library Stdlib.ZArith.BinInt

-

Specification of comparisons and order

+

Specification of comparisons and order

@@ -588,7 +588,7 @@

Library Stdlib.ZArith.BinInt

-

Specification of minimum and maximum

+

Specification of minimum and maximum

@@ -609,7 +609,7 @@

Library Stdlib.ZArith.BinInt

-

Induction principles based on successor / predecessor

+

Induction principles based on successor / predecessor

@@ -650,7 +650,7 @@

Library Stdlib.ZArith.BinInt

-

Specification of absolute value

+

Specification of absolute value

@@ -665,7 +665,7 @@

Library Stdlib.ZArith.BinInt

-

Specification of sign

+

Specification of sign

@@ -683,7 +683,7 @@

Library Stdlib.ZArith.BinInt

-

Specification of power

+

Specification of power

@@ -712,7 +712,7 @@

Library Stdlib.ZArith.BinInt

-

Specification of square

+

Specification of square

@@ -724,7 +724,7 @@

Library Stdlib.ZArith.BinInt

-

Specification of square root

+

Specification of square root

@@ -747,7 +747,7 @@

Library Stdlib.ZArith.BinInt

-

Specification of logarithm

+

Specification of logarithm

@@ -776,7 +776,7 @@

Library Stdlib.ZArith.BinInt

-

Multiplication and Doubling

+

Multiplication and Doubling

@@ -794,7 +794,7 @@

Library Stdlib.ZArith.BinInt

-

Correctness proofs for Trunc division

+

Correctness proofs for Trunc division

@@ -826,7 +826,7 @@

Library Stdlib.ZArith.BinInt

-

Correctness proofs for Floor division

+

Correctness proofs for Floor division

@@ -859,7 +859,7 @@

Library Stdlib.ZArith.BinInt

-

Extra properties about divide

+

Extra properties about divide

@@ -877,7 +877,7 @@

Library Stdlib.ZArith.BinInt

-

Correctness proofs for gcd

+

Correctness proofs for gcd

@@ -918,7 +918,7 @@

Library Stdlib.ZArith.BinInt

-

Extra properties about testbit

+

Extra properties about testbit

@@ -943,7 +943,7 @@

Library Stdlib.ZArith.BinInt

-

Proofs of specifications for bitwise operations

+

Proofs of specifications for bitwise operations

@@ -1122,7 +1122,7 @@

Library Stdlib.ZArith.BinInt

-

Comparison and opposite

+

Comparison and opposite

@@ -1134,7 +1134,7 @@

Library Stdlib.ZArith.BinInt

-

Comparison and addition

+

Comparison and addition

@@ -1146,7 +1146,7 @@

Library Stdlib.ZArith.BinInt

-

testbit in terms of comparison.

+

testbit in terms of comparison.

diff --git a/master/stdlib/Stdlib.ZArith.BinIntDef.html b/master/stdlib/Stdlib.ZArith.BinIntDef.html index a641787121..d613ac06a7 100644 --- a/master/stdlib/Stdlib.ZArith.BinIntDef.html +++ b/master/stdlib/Stdlib.ZArith.BinIntDef.html @@ -61,7 +61,7 @@

Library Stdlib.ZArith.BinIntDef

-

Binary Integers, Definitions of Operations

+

Binary Integers, Definitions of Operations

@@ -79,7 +79,7 @@

Library Stdlib.ZArith.BinIntDef

-

Nicer names Z.pos and Z.neg for constructors

+

Nicer names Z.pos and Z.neg for constructors

@@ -92,7 +92,7 @@

Library Stdlib.ZArith.BinIntDef

-

Constants

+

Constants

@@ -106,7 +106,7 @@

Library Stdlib.ZArith.BinIntDef

-

Doubling and variants

+

Doubling and variants

@@ -139,7 +139,7 @@

Library Stdlib.ZArith.BinIntDef

-

Subtraction of positive into Z

+

Subtraction of positive into Z

@@ -162,7 +162,7 @@

Library Stdlib.ZArith.BinIntDef

-

Addition

+

Addition

@@ -185,7 +185,7 @@

Library Stdlib.ZArith.BinIntDef

-

Opposite

+

Opposite

@@ -205,7 +205,7 @@

Library Stdlib.ZArith.BinIntDef

-

Successor

+

Successor

@@ -217,7 +217,7 @@

Library Stdlib.ZArith.BinIntDef

-

Predecessor

+

Predecessor

@@ -229,7 +229,7 @@

Library Stdlib.ZArith.BinIntDef

-

Subtraction

+

Subtraction

@@ -244,7 +244,7 @@

Library Stdlib.ZArith.BinIntDef

-

Multiplication

+

Multiplication

@@ -267,7 +267,7 @@

Library Stdlib.ZArith.BinIntDef

-

Power function

+

Power function

@@ -290,7 +290,7 @@

Library Stdlib.ZArith.BinIntDef

-

Square

+

Square

@@ -307,7 +307,7 @@

Library Stdlib.ZArith.BinIntDef

-

Comparison

+

Comparison

@@ -333,7 +333,7 @@

Library Stdlib.ZArith.BinIntDef

-

Sign function

+

Sign function

@@ -412,7 +412,7 @@

Library Stdlib.ZArith.BinIntDef

-

Minimum and maximum

+

Minimum and maximum

@@ -435,7 +435,7 @@

Library Stdlib.ZArith.BinIntDef

-

Absolute value

+

Absolute value

@@ -452,7 +452,7 @@

Library Stdlib.ZArith.BinIntDef

-

Conversions

+

Conversions

@@ -627,7 +627,7 @@

Library Stdlib.ZArith.BinIntDef

-

Iteration of a function

+

Iteration of a function

@@ -648,7 +648,7 @@

Library Stdlib.ZArith.BinIntDef

-

Euclidean divisions for binary integers

+

Euclidean divisions for binary integers

@@ -663,7 +663,7 @@

Library Stdlib.ZArith.BinIntDef

-

Floor division

+

Floor division

@@ -758,7 +758,7 @@

Library Stdlib.ZArith.BinIntDef

-

Trunc Division

+

Trunc Division

@@ -819,7 +819,7 @@

Library Stdlib.ZArith.BinIntDef

No infix notation for rem, otherwise it becomes a keyword
-

Parity functions

+

Parity functions

@@ -846,7 +846,7 @@

Library Stdlib.ZArith.BinIntDef

-

Division by two

+

Division by two

@@ -892,7 +892,7 @@

Library Stdlib.ZArith.BinIntDef

NB: Z.quot2 used to be named Z.div2 in Coq <= 8.3
-

Base-2 logarithm

+

Base-2 logarithm

@@ -909,7 +909,7 @@

Library Stdlib.ZArith.BinIntDef

-

Square root

+

Square root

@@ -937,7 +937,7 @@

Library Stdlib.ZArith.BinIntDef

-

Greatest Common Divisor

+

Greatest Common Divisor

@@ -980,7 +980,7 @@

Library Stdlib.ZArith.BinIntDef

-

Bitwise functions

+

Bitwise functions

diff --git a/master/stdlib/Stdlib.ZArith.Int.html b/master/stdlib/Stdlib.ZArith.Int.html index 183f1561fa..2d21e20869 100644 --- a/master/stdlib/Stdlib.ZArith.Int.html +++ b/master/stdlib/Stdlib.ZArith.Int.html @@ -49,7 +49,7 @@

Library Stdlib.ZArith.Int

-

An light axiomatization of integers (used in MSetAVL).

+

An light axiomatization of integers (used in MSetAVL).

@@ -74,7 +74,7 @@

Library Stdlib.ZArith.Int

-

A specification of integers

+

A specification of integers

@@ -210,7 +210,7 @@

Library Stdlib.ZArith.Int

-

Facts and tactics using Int

+

Facts and tactics using Int

@@ -564,7 +564,7 @@

Library Stdlib.ZArith.Int

-

An implementation of Int

+

An implementation of Int

diff --git a/master/stdlib/Stdlib.ZArith.ZArith_dec.html b/master/stdlib/Stdlib.ZArith.ZArith_dec.html index f5536e1d8f..7605d48beb 100644 --- a/master/stdlib/Stdlib.ZArith.ZArith_dec.html +++ b/master/stdlib/Stdlib.ZArith.ZArith_dec.html @@ -74,7 +74,7 @@

Library Stdlib.ZArith.ZArith_dec

-

Decidability of order on binary integers

+

Decidability of order on binary integers

@@ -116,7 +116,7 @@

Library Stdlib.ZArith.ZArith_dec

-

Cotransitivity of order on binary integers

+

Cotransitivity of order on binary integers

diff --git a/master/stdlib/Stdlib.ZArith.Zabs.html b/master/stdlib/Stdlib.ZArith.Zabs.html index a551923faf..8cbd850857 100644 --- a/master/stdlib/Stdlib.ZArith.Zabs.html +++ b/master/stdlib/Stdlib.ZArith.Zabs.html @@ -74,7 +74,7 @@

Library Stdlib.ZArith.Zabs

-

Properties of absolute value

+

Properties of absolute value

@@ -92,7 +92,7 @@

Library Stdlib.ZArith.Zabs

-

Proving a property of the absolute value by cases

+

Proving a property of the absolute value by cases

@@ -117,7 +117,7 @@

Library Stdlib.ZArith.Zabs

-

Some results about the sign function.

+

Some results about the sign function.

diff --git a/master/stdlib/Stdlib.ZArith.Zbitwise.html b/master/stdlib/Stdlib.ZArith.Zbitwise.html index d84d113dfc..9a476c2c29 100644 --- a/master/stdlib/Stdlib.ZArith.Zbitwise.html +++ b/master/stdlib/Stdlib.ZArith.Zbitwise.html @@ -152,13 +152,13 @@

Library Stdlib.ZArith.Zbitwise

Explicit formulas for carry bits during addition. Conceptually, the theory -

here matches the bitblasting rules for integers. However, the vector of

+

here matches the bitblasting rules for integers. However, the vector of

-

carry bits is represented as a Z so it can be used in bitwise operations.

+

carry bits is represented as a Z so it can be used in bitwise operations.

-

The last three lemmas about addcarries are the main interface, but the

+

The last three lemmas about addcarries are the main interface, but the

-

generalization adccarries is provided as the same theory applies.

+

generalization adccarries is provided as the same theory applies.

diff --git a/master/stdlib/Stdlib.ZArith.Zbool.html b/master/stdlib/Stdlib.ZArith.Zbool.html index 005b5c0668..b3f9e6d1bf 100644 --- a/master/stdlib/Stdlib.ZArith.Zbool.html +++ b/master/stdlib/Stdlib.ZArith.Zbool.html @@ -60,7 +60,7 @@

Library Stdlib.ZArith.Zbool

-

Boolean operations from decidability of order

+

Boolean operations from decidability of order

The decidability of equality and order relations over type Z gives some boolean functions with the adequate specification.
@@ -85,7 +85,7 @@

Library Stdlib.ZArith.Zbool

-

Boolean comparisons of binary integers

+

Boolean comparisons of binary integers

diff --git a/master/stdlib/Stdlib.ZArith.Zcompare.html b/master/stdlib/Stdlib.ZArith.Zcompare.html index bbdc04e4cf..d557491763 100644 --- a/master/stdlib/Stdlib.ZArith.Zcompare.html +++ b/master/stdlib/Stdlib.ZArith.Zcompare.html @@ -68,7 +68,7 @@

Library Stdlib.ZArith.Zcompare

-

Comparison on integers

+

Comparison on integers

@@ -83,7 +83,7 @@

Library Stdlib.ZArith.Zcompare

-

Transitivity of comparison

+

Transitivity of comparison

@@ -100,7 +100,7 @@

Library Stdlib.ZArith.Zcompare

-

Comparison and opposite

+

Comparison and opposite

@@ -112,7 +112,7 @@

Library Stdlib.ZArith.Zcompare

-

Comparison first-order specification

+

Comparison first-order specification

@@ -124,7 +124,7 @@

Library Stdlib.ZArith.Zcompare

-

Comparison and addition

+

Comparison and addition

@@ -146,7 +146,7 @@

Library Stdlib.ZArith.Zcompare

-

Successor and comparison

+

Successor and comparison

@@ -158,7 +158,7 @@

Library Stdlib.ZArith.Zcompare

-

Multiplication and comparison

+

Multiplication and comparison

@@ -179,7 +179,7 @@

Library Stdlib.ZArith.Zcompare

-

Relating x ?= y to =, <=, <, >= or >

+

Relating x ?= y to =, <=, <, >= or >

diff --git a/master/stdlib/Stdlib.ZArith.Zdiv.html b/master/stdlib/Stdlib.ZArith.Zdiv.html index d6833676b9..88589b7763 100644 --- a/master/stdlib/Stdlib.ZArith.Zdiv.html +++ b/master/stdlib/Stdlib.ZArith.Zdiv.html @@ -49,7 +49,7 @@

Library Stdlib.ZArith.Zdiv

-

Euclidean Division

+

Euclidean Division

@@ -89,7 +89,7 @@

Library Stdlib.ZArith.Zdiv

-

Main division theorems

+

Main division theorems

@@ -238,7 +238,7 @@

Library Stdlib.ZArith.Zdiv

-

Basic values of divisions and modulo.

+

Basic values of divisions and modulo.

@@ -294,7 +294,7 @@

Library Stdlib.ZArith.Zdiv

-

Order results about Z.modulo and Z.div

+

Order results about Z.modulo and Z.div

@@ -452,7 +452,7 @@

Library Stdlib.ZArith.Zdiv

-

Relations between usual operations and Z.modulo and Z.div

+

Relations between usual operations and Z.modulo and Z.div

@@ -691,7 +691,7 @@

Library Stdlib.ZArith.Zdiv

-

Compatibility

+

Compatibility

@@ -727,7 +727,7 @@

Library Stdlib.ZArith.Zdiv

-

A direct way to compute Z.modulo

+

A direct way to compute Z.modulo

@@ -779,9 +779,9 @@

Library Stdlib.ZArith.Zdiv

Another convention is possible for division by negative numbers: -

quotient is always the biggest integer smaller than or equal to a/b

+

quotient is always the biggest integer smaller than or equal to a/b

-

remainder is hence always positive or null.

+

remainder is hence always positive or null.

diff --git a/master/stdlib/Stdlib.ZArith.Zeuclid.html b/master/stdlib/Stdlib.ZArith.Zeuclid.html index d5c68f2429..c3064ca1dd 100644 --- a/master/stdlib/Stdlib.ZArith.Zeuclid.html +++ b/master/stdlib/Stdlib.ZArith.Zeuclid.html @@ -63,7 +63,7 @@

Library Stdlib.ZArith.Zeuclid

-

Definitions of division for binary integers, Euclid convention.

+

Definitions of division for binary integers, Euclid convention.

diff --git a/master/stdlib/Stdlib.ZArith.Zeven.html b/master/stdlib/Stdlib.ZArith.Zeven.html index e6b1d3cf5c..9f4268d1fc 100644 --- a/master/stdlib/Stdlib.ZArith.Zeven.html +++ b/master/stdlib/Stdlib.ZArith.Zeven.html @@ -176,7 +176,7 @@

Library Stdlib.ZArith.Zeven

-

Definition of Z.quot2, Z.div2 and properties wrt Zeven

+

Definition of Z.quot2, Z.div2 and properties wrt Zeven

and Zodd
diff --git a/master/stdlib/Stdlib.ZArith.Zgcd_alt.html b/master/stdlib/Stdlib.ZArith.Zgcd_alt.html index ea77ec79d7..16dfc51ac9 100644 --- a/master/stdlib/Stdlib.ZArith.Zgcd_alt.html +++ b/master/stdlib/Stdlib.ZArith.Zgcd_alt.html @@ -49,7 +49,7 @@

Library Stdlib.ZArith.Zgcd_alt

-

Zgcd_alt : an alternate version of Z.gcd, based on Euclid's algorithm

+

Zgcd_alt : an alternate version of Z.gcd, based on Euclid's algorithm

diff --git a/master/stdlib/Stdlib.ZArith.Zhints.html b/master/stdlib/Stdlib.ZArith.Zhints.html index 315d14ce01..681c317c44 100644 --- a/master/stdlib/Stdlib.ZArith.Zhints.html +++ b/master/stdlib/Stdlib.ZArith.Zhints.html @@ -102,7 +102,7 @@

Library Stdlib.ZArith.Zhints

-

Simplification lemmas

+

Simplification lemmas

@@ -116,7 +116,7 @@

Library Stdlib.ZArith.Zhints

  
-

Reversible simplification lemmas (no loss of information)

+

Reversible simplification lemmas (no loss of information)

Should clearly be declared as hints
@@ -171,7 +171,7 @@

Library Stdlib.ZArith.Zhints

  
-

Irreversible simplification lemmas

+

Irreversible simplification lemmas

Probably to be declared as hints, when no other simplification is possible
diff --git a/master/stdlib/Stdlib.ZArith.Znat.html b/master/stdlib/Stdlib.ZArith.Znat.html index ab4a9c7016..0987053f0e 100644 --- a/master/stdlib/Stdlib.ZArith.Znat.html +++ b/master/stdlib/Stdlib.ZArith.Znat.html @@ -95,7 +95,7 @@

Library Stdlib.ZArith.Znat

-

Chains of conversions

+

Chains of conversions

@@ -148,7 +148,7 @@

Library Stdlib.ZArith.Znat

-

Conversions between Z and N

+

Conversions between Z and N

@@ -552,7 +552,7 @@

Library Stdlib.ZArith.Znat

-

Conversions between Z and nat

+

Conversions between Z and nat

diff --git a/master/stdlib/Stdlib.ZArith.Znumtheory.html b/master/stdlib/Stdlib.ZArith.Znumtheory.html index bb50c51117..54bed36175 100644 --- a/master/stdlib/Stdlib.ZArith.Znumtheory.html +++ b/master/stdlib/Stdlib.ZArith.Znumtheory.html @@ -245,7 +245,7 @@

Library Stdlib.ZArith.Znumtheory

-

Greatest common divisor (gcd).

+

Greatest common divisor (gcd).

@@ -307,7 +307,7 @@

Library Stdlib.ZArith.Znumtheory

-

Extended Euclid algorithm.

+

Extended Euclid algorithm.

@@ -395,7 +395,7 @@

Library Stdlib.ZArith.Znumtheory

-

Bezout's coefficients

+

Bezout's coefficients

@@ -431,7 +431,7 @@

Library Stdlib.ZArith.Znumtheory

-

Relative primality

+

Relative primality

@@ -525,7 +525,7 @@

Library Stdlib.ZArith.Znumtheory

-

Primality

+

Primality

diff --git a/master/stdlib/Stdlib.ZArith.Zorder.html b/master/stdlib/Stdlib.ZArith.Zorder.html index ca3986a24d..8256f7e3fe 100644 --- a/master/stdlib/Stdlib.ZArith.Zorder.html +++ b/master/stdlib/Stdlib.ZArith.Zorder.html @@ -71,7 +71,7 @@

Library Stdlib.ZArith.Zorder

Properties of the order relations on binary integers
-

Trichotomy

+

Trichotomy

@@ -86,7 +86,7 @@

Library Stdlib.ZArith.Zorder

-

Decidability of equality and order on Z

+

Decidability of equality and order on Z

@@ -112,7 +112,7 @@

Library Stdlib.ZArith.Zorder

-

Relating strict and large orders

+

Relating strict and large orders

@@ -152,7 +152,7 @@

Library Stdlib.ZArith.Zorder

-

Equivalence and order properties

+

Equivalence and order properties

@@ -276,11 +276,11 @@

Library Stdlib.ZArith.Zorder

-

Compatibility of order and operations on Z

+

Compatibility of order and operations on Z

-

Successor

+

Successor

@@ -458,7 +458,7 @@

Library Stdlib.ZArith.Zorder

-

Addition

+

Addition

Compatibility of addition wrt to order
@@ -528,7 +528,7 @@

Library Stdlib.ZArith.Zorder

-

Multiplication

+

Multiplication

Compatibility of multiplication by a positive wrt to order
@@ -656,7 +656,7 @@

Library Stdlib.ZArith.Zorder

-

Square

+

Square

Simplification of square wrt order
@@ -671,7 +671,7 @@

Library Stdlib.ZArith.Zorder

-

Equivalence between inequalities

+

Equivalence between inequalities

diff --git a/master/stdlib/Stdlib.ZArith.Zpow_def.html b/master/stdlib/Stdlib.ZArith.Zpow_def.html index 3ba3dbf84f..a467567a9e 100644 --- a/master/stdlib/Stdlib.ZArith.Zpow_def.html +++ b/master/stdlib/Stdlib.ZArith.Zpow_def.html @@ -53,7 +53,7 @@

Library Stdlib.ZArith.Zpow_def

-

Power functions over Z

+

Power functions over Z

diff --git a/master/stdlib/Stdlib.ZArith.Zpow_facts.html b/master/stdlib/Stdlib.ZArith.Zpow_facts.html index 097409c0c1..96b57e7a07 100644 --- a/master/stdlib/Stdlib.ZArith.Zpow_facts.html +++ b/master/stdlib/Stdlib.ZArith.Zpow_facts.html @@ -132,7 +132,7 @@

Library Stdlib.ZArith.Zpow_facts

-

Z.pow and modulo

+

Z.pow and modulo

@@ -208,7 +208,7 @@

Library Stdlib.ZArith.Zpow_facts

-

Z.square: a direct definition of z^2

+

Z.square: a direct definition of z^2

diff --git a/master/stdlib/Stdlib.ZArith.Zpower.html b/master/stdlib/Stdlib.ZArith.Zpower.html index 66f3bc1ab9..e7eec2e0b1 100644 --- a/master/stdlib/Stdlib.ZArith.Zpower.html +++ b/master/stdlib/Stdlib.ZArith.Zpower.html @@ -54,7 +54,7 @@

Library Stdlib.ZArith.Zpower

-

Power functions over Z

+

Power functions over Z

@@ -154,7 +154,7 @@

Library Stdlib.ZArith.Zpower

-

Powers of 2

+

Powers of 2

@@ -283,7 +283,7 @@

Library Stdlib.ZArith.Zpower

-

Division by a power of two.

+

Division by a power of two.

diff --git a/master/stdlib/Stdlib.ZArith.Zquot.html b/master/stdlib/Stdlib.ZArith.Zquot.html index 4e76b92015..2ef5e49a53 100644 --- a/master/stdlib/Stdlib.ZArith.Zquot.html +++ b/master/stdlib/Stdlib.ZArith.Zquot.html @@ -153,7 +153,7 @@

Library Stdlib.ZArith.Zquot

-

Division and Opposite

+

Division and Opposite

@@ -232,7 +232,7 @@

Library Stdlib.ZArith.Zquot

-

Unicity results

+

Unicity results

@@ -265,7 +265,7 @@

Library Stdlib.ZArith.Zquot

-

Order results about Zrem and Zquot

+

Order results about Zrem and Zquot

@@ -363,7 +363,7 @@

Library Stdlib.ZArith.Zquot

-

Relations between usual operations and Z.modulo and Z.div

+

Relations between usual operations and Z.modulo and Z.div

@@ -527,7 +527,7 @@

Library Stdlib.ZArith.Zquot

-

Interaction with "historic" Zdiv

+

Interaction with "historic" Zdiv

diff --git a/master/stdlib/Stdlib.ZArith.auxiliary.html b/master/stdlib/Stdlib.ZArith.auxiliary.html index fc5abca2f2..8394ab43e5 100644 --- a/master/stdlib/Stdlib.ZArith.auxiliary.html +++ b/master/stdlib/Stdlib.ZArith.auxiliary.html @@ -68,7 +68,7 @@

Library Stdlib.ZArith.auxiliary

-

Moving terms from one side to the other of an inequality

+

Moving terms from one side to the other of an inequality

diff --git a/master/stdlib/Stdlib.btauto.Algebra.html b/master/stdlib/Stdlib.btauto.Algebra.html index b8b0b108a4..4806d3c624 100644 --- a/master/stdlib/Stdlib.btauto.Algebra.html +++ b/master/stdlib/Stdlib.btauto.Algebra.html @@ -144,7 +144,7 @@

Library Stdlib.btauto.Algebra

-

Global, inductive definitions.

+

Global, inductive definitions.

@@ -217,7 +217,7 @@

Library Stdlib.btauto.Algebra

-

The core reflexive part.

+

The core reflexive part.

diff --git a/master/stdlib/Stdlib.extraction.ExtrHaskellNatInt.html b/master/stdlib/Stdlib.extraction.ExtrHaskellNatInt.html index 12f2636194..aedbc70272 100644 --- a/master/stdlib/Stdlib.extraction.ExtrHaskellNatInt.html +++ b/master/stdlib/Stdlib.extraction.ExtrHaskellNatInt.html @@ -62,11 +62,11 @@

Library Stdlib.extraction.ExtrHaskellNatInt

-

Disclaimer: trying to obtain efficient certified programs

+

Disclaimer: trying to obtain efficient certified programs

-

by extracting nat into Int is definitively *not* a good idea.

+

by extracting nat into Int is definitively *not* a good idea.

-

See comments in ExtrOcamlNatInt.v.

+

See comments in ExtrOcamlNatInt.v.

diff --git a/master/stdlib/Stdlib.extraction.ExtrHaskellNatInteger.html b/master/stdlib/Stdlib.extraction.ExtrHaskellNatInteger.html index 1e98eec322..1aaaac09f0 100644 --- a/master/stdlib/Stdlib.extraction.ExtrHaskellNatInteger.html +++ b/master/stdlib/Stdlib.extraction.ExtrHaskellNatInteger.html @@ -62,11 +62,11 @@

Library Stdlib.extraction.ExtrHaskellNatInteger

-

Disclaimer: trying to obtain efficient certified programs

+

Disclaimer: trying to obtain efficient certified programs

-

by extracting nat into Integer isn't necessarily a good idea.

+

by extracting nat into Integer isn't necessarily a good idea.

-

See comments in ExtrOcamlNatInt.v.

+

See comments in ExtrOcamlNatInt.v.

diff --git a/master/stdlib/Stdlib.extraction.ExtrHaskellNatNum.html b/master/stdlib/Stdlib.extraction.ExtrHaskellNatNum.html index 21b5aa9698..67e640ec1d 100644 --- a/master/stdlib/Stdlib.extraction.ExtrHaskellNatNum.html +++ b/master/stdlib/Stdlib.extraction.ExtrHaskellNatNum.html @@ -47,15 +47,15 @@

Library Stdlib.extraction.ExtrHaskellNatNum

-

Efficient (but uncertified) extraction of usual nat functions

+

Efficient (but uncertified) extraction of usual nat functions

-

into equivalent versions in Haskell's Prelude that are defined

+

into equivalent versions in Haskell's Prelude that are defined

-

for any Num typeclass instances. Useful in combination with

+

for any Num typeclass instances. Useful in combination with

-

Extract Inductive nat that maps nat onto a Haskell type that

+

Extract Inductive nat that maps nat onto a Haskell type that

-

implements Num.

+

implements Num.

diff --git a/master/stdlib/Stdlib.extraction.ExtrHaskellString.html b/master/stdlib/Stdlib.extraction.ExtrHaskellString.html index dcf302b855..850f895a9f 100644 --- a/master/stdlib/Stdlib.extraction.ExtrHaskellString.html +++ b/master/stdlib/Stdlib.extraction.ExtrHaskellString.html @@ -47,7 +47,7 @@

Library Stdlib.extraction.ExtrHaskellString

-

Special handling of ascii and strings for extraction to Haskell.

+

Special handling of ascii and strings for extraction to Haskell.

@@ -68,16 +68,16 @@

Library Stdlib.extraction.ExtrHaskellString

-

At the moment, Coq's extraction has no way to add extra import

+

At the moment, Coq's extraction has no way to add extra import

-

statements to the extracted Haskell code. You will have to

+

statements to the extracted Haskell code. You will have to

-

manually add:

+

manually add:

* -

import qualified Data.Bits

+

import qualified Data.Bits

-

import qualified Data.Char

+

import qualified Data.Char

diff --git a/master/stdlib/Stdlib.extraction.ExtrHaskellZInt.html b/master/stdlib/Stdlib.extraction.ExtrHaskellZInt.html index 5d4dc06044..1c0e03d5c3 100644 --- a/master/stdlib/Stdlib.extraction.ExtrHaskellZInt.html +++ b/master/stdlib/Stdlib.extraction.ExtrHaskellZInt.html @@ -62,11 +62,11 @@

Library Stdlib.extraction.ExtrHaskellZInt

-

Disclaimer: trying to obtain efficient certified programs

+

Disclaimer: trying to obtain efficient certified programs

-

by extracting Z into Int is definitively *not* a good idea.

+

by extracting Z into Int is definitively *not* a good idea.

-

See comments in ExtrOcamlNatInt.v.

+

See comments in ExtrOcamlNatInt.v.

diff --git a/master/stdlib/Stdlib.extraction.ExtrHaskellZNum.html b/master/stdlib/Stdlib.extraction.ExtrHaskellZNum.html index 16b579dc2e..7ab2f3cd97 100644 --- a/master/stdlib/Stdlib.extraction.ExtrHaskellZNum.html +++ b/master/stdlib/Stdlib.extraction.ExtrHaskellZNum.html @@ -47,15 +47,15 @@

Library Stdlib.extraction.ExtrHaskellZNum

-

Efficient (but uncertified) extraction of usual Z functions

+

Efficient (but uncertified) extraction of usual Z functions

-

into equivalent versions in Haskell's Prelude that are defined

+

into equivalent versions in Haskell's Prelude that are defined

-

for any Num typeclass instances. Useful in combination with

+

for any Num typeclass instances. Useful in combination with

-

Extract Inductive Z that maps Z onto a Haskell type that

+

Extract Inductive Z that maps Z onto a Haskell type that

-

implements Num.

+

implements Num.

diff --git a/master/stdlib/Stdlib.omega.PreOmega.html b/master/stdlib/Stdlib.omega.PreOmega.html index aec7577fba..bda124fd90 100644 --- a/master/stdlib/Stdlib.omega.PreOmega.html +++ b/master/stdlib/Stdlib.omega.PreOmega.html @@ -55,7 +55,7 @@

Library Stdlib.omega.PreOmega

-

Z.div_mod_to_equations, Z.quot_rem_to_equations, Z.to_euclidean_division_equations:

+

Z.div_mod_to_equations, Z.quot_rem_to_equations, Z.to_euclidean_division_equations:

the tactics for preprocessing Z.div and Z.modulo, Z.quot and Z.rem
diff --git a/master/stdlib/index_global_B.html b/master/stdlib/index_global_B.html index 90b329ad43..75a664857c 100644 --- a/master/stdlib/index_global_B.html +++ b/master/stdlib/index_global_B.html @@ -1014,8 +1014,8 @@ BVor [definition, in Stdlib.Bool.Bvector]
BVxor [definition, in Stdlib.Bool.Bvector]
byte [inductive, in Stdlib.Init.Byte]
-Byte [library]
Byte [library]
+Byte [library]
ByteNotations [module, in Stdlib.Strings.Byte]
_ =? _ (byte_scope) [notation, in Stdlib.Strings.Byte]
ByteSyntaxNotations [module, in Stdlib.Init.Byte]
diff --git a/master/stdlib/index_global_T.html b/master/stdlib/index_global_T.html index f82d22a000..39fa7d19d2 100644 --- a/master/stdlib/index_global_T.html +++ b/master/stdlib/index_global_T.html @@ -529,8 +529,8 @@ t [inductive, in Stdlib.Vectors.Fin]
t [definition, in Stdlib.Init.Nat]
t [inductive, in Stdlib.Vectors.VectorDef]
-Tactics [library]
Tactics [library]
+Tactics [library]
tactic_view [constructor, in Stdlib.ssr.ssreflect]
Tadd [definition, in Stdlib.rtauto.Bintree]
tag [definition, in Stdlib.ssr.ssrfun]
@@ -598,8 +598,8 @@ tan_plus [lemma, in Stdlib.Reals.Rtrigo1]
target [projection, in Stdlib.micromega.ZifyClasses]
target_prop [projection, in Stdlib.micromega.ZifyClasses]
-Tauto [library]
Tauto [library]
+Tauto [library]
tauto_checker_sound [lemma, in Stdlib.micromega.Tauto]
tauto_checker [definition, in Stdlib.micromega.Tauto]
TBOp [projection, in Stdlib.micromega.ZifyClasses]
diff --git a/master/stdlib/index_global_W.html b/master/stdlib/index_global_W.html index 0b8cdccd3a..179d9e83e1 100644 --- a/master/stdlib/index_global_W.html +++ b/master/stdlib/index_global_W.html @@ -958,8 +958,8 @@ WEqProperties_fun.Add [definition, in Stdlib.FSets.FSetEqProperties]
WEqProperties_fun.MP [module, in Stdlib.FSets.FSetEqProperties]
WEqProperties_fun [module, in Stdlib.FSets.FSetEqProperties]
-Wf [library]
Wf [library]
+Wf [library]
WFacts [module, in Stdlib.FSets.FMapFacts]
WFacts [module, in Stdlib.FSets.FSetFacts]
WFacts [module, in Stdlib.MSets.MSetFacts]
diff --git a/master/stdlib/index_library_B.html b/master/stdlib/index_library_B.html index d4a21d2461..0442aa8988 100644 --- a/master/stdlib/index_library_B.html +++ b/master/stdlib/index_library_B.html @@ -545,8 +545,8 @@ Bool_nat
Btauto
Bvector
-Byte
Byte
+Byte