coqide-server.protocol
Serialize
btauto_plugin
cc_plugin
coq-core.clib
coq-core.config
coq-core.engine
coq-core.gramlib
coq-core.interp
coq-core.kernel
coq-core.lib
coq-core.library
coq-core.parsing
coq-core.plugins
coq-core.pretyping
coq-core.printing
coq-core.proofs
coq-core.stm
coq-core.sysinit
coq-core.tactics
coq-core.top_printers
coq-core.toplevel
coq-core.vernac
coq-core.vm
coqide-server.core
derive_plugin
extraction_plugin
firstorder_plugin
float_syntax_plugin
funind_plugin
ltac2_plugin
ltac_plugin
micromega_plugin
nsatz_plugin
number_string_notation_plugin
ring_plugin
rtauto_plugin
ssreflect_plugin
ssrmatching_plugin
ssrsearch_plugin
tauto_plugin
tuto0_plugin
tuto1_plugin
tuto2_plugin
tuto3_plugin
zify_plugin
exception Marshal_error of string * Xml_datatype.xml
val massoc : string -> (string * string) list -> string
val constructor : string -> string -> Xml_datatype.xml list -> Xml_datatype.xml
val do_match : string -> (string -> Xml_datatype.xml list -> 'b) -> Xml_datatype.xml -> 'b
val singleton : 'a list -> 'a
val empty : 'a list -> unit
val raw_string : Xml_datatype.xml list -> string
val of_unit : unit -> Xml_datatype.xml
val to_unit : Xml_datatype.xml -> unit
val of_bool : bool -> Xml_datatype.xml
val to_bool : Xml_datatype.xml -> bool
val of_list : ('a -> Xml_datatype.xml) -> 'a list -> Xml_datatype.xml
val to_list : (Xml_datatype.xml -> 'a) -> Xml_datatype.xml -> 'a list
val of_option : ('a -> Xml_datatype.xml) -> 'a option -> Xml_datatype.xml
val to_option : (Xml_datatype.xml -> 'a) -> Xml_datatype.xml -> 'a option
val of_string : string -> Xml_datatype.xml
val to_string : Xml_datatype.xml -> string
val of_int : int -> Xml_datatype.xml
val to_int : Xml_datatype.xml -> int
val of_pair : ('a -> Xml_datatype.xml) -> ('b -> Xml_datatype.xml) -> ('a * 'b) -> Xml_datatype.xml
val to_pair : (Xml_datatype.xml -> 'a) -> (Xml_datatype.xml -> 'b) -> Xml_datatype.xml -> 'a * 'b
val of_union : ('a -> Xml_datatype.xml) -> ('b -> Xml_datatype.xml) -> ('a, 'b) CSig.union -> Xml_datatype.xml
val to_union : (Xml_datatype.xml -> 'a) -> (Xml_datatype.xml -> 'b) -> Xml_datatype.xml -> ('a, 'b) CSig.union
val of_edit_id : int -> Xml_datatype.xml
val to_edit_id : Xml_datatype.xml -> int
val of_loc : Loc.t -> Xml_datatype.xml
val to_loc : Xml_datatype.xml -> Loc.t
val of_xml : Xml_datatype.xml -> Xml_datatype.xml
val to_xml : Xml_datatype.xml -> Xml_datatype.xml