package coq
 sectionYPositions = computeSectionYPositions($el), 10)"
  x-init="setTimeout(() => sectionYPositions = computeSectionYPositions($el), 10)"
  >
  
  
  Formal proof management system
Install
    
    dune-project
 Dependency
Authors
Maintainers
Sources
  
    
      coq-8.14.1.tar.gz
    
    
        
    
  
  
  
    
  
        sha256=3cbfc1e1a72b16d4744f5b64ede59586071e31d9c11c811a0372060727bfd9c3
    
    
  doc/firstorder_plugin/Firstorder_plugin/Formula/index.html
Module Firstorder_plugin.FormulaSource
Source
val (==?) : 
  ('a -> 'a -> 'b -> 'b -> int) ->
  ('c -> 'c -> int) ->
  'a ->
  'a ->
  'b ->
  'b ->
  'c ->
  'c ->
  intSource
val ind_hyps : 
  Environ.env ->
  Evd.evar_map ->
  int ->
  Constr.pinductive ->
  EConstr.constr list ->
  EConstr.rel_context arraySource
val build_atoms : 
  Environ.env ->
  Evd.evar_map ->
  counter ->
  side ->
  EConstr.constr ->
  bool * atomsSource
type right_pattern = - | Rarrow
- | Rand
- | Ror
- | Rfalse
- | Rforall
- | Rexists of Constr.metavariable * EConstr.constr * bool
Source
type left_arrow_pattern = - | LLatom
- | LLfalse of Constr.pinductive * EConstr.constr list
- | LLand of Constr.pinductive * EConstr.constr list
- | LLor of Constr.pinductive * EConstr.constr list
- | LLforall of EConstr.constr
- | LLexists of Constr.pinductive * EConstr.constr list
- | LLarrow of EConstr.constr * EConstr.constr * EConstr.constr
Source
type left_pattern = - | Lfalse
- | Land of Constr.pinductive
- | Lor of Constr.pinductive
- | Lforall of Constr.metavariable * EConstr.constr * bool
- | Lexists of Constr.pinductive
- | LA of EConstr.constr * left_arrow_pattern
Source
type t = {- id : Names.GlobRef.t;
- constr : EConstr.constr;
- pat : (left_pattern, right_pattern) sum;
- atoms : atoms;
}Source
val build_formula : 
  Environ.env ->
  Evd.evar_map ->
  side ->
  Names.GlobRef.t ->
  EConstr.types ->
  counter ->
  (t, EConstr.types) sum sectionYPositions = computeSectionYPositions($el), 10)"
  x-init="setTimeout(() => sectionYPositions = computeSectionYPositions($el), 10)"
  >