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.15.2.tar.gz
    
    
        
    
  
  
  
    
  
        sha256=13a67c0a4559ae22e9765c8fdb88957b16c2b335a2d5f47e4d6d9b4b8b299926
    
    
  doc/cc_plugin/Cc_plugin/Ccproof/index.html
Module Cc_plugin.CcproofSource
Source
type rule = - | Ax of Constr.constr
- | SymAx of Constr.constr
- | Refl of Ccalgo.ATerm.t
- | Trans of proof * proof
- | Congr of proof * proof
- | Inject of proof * Constr.pconstructor * int * int
Proof smart constructors
Source
val pax : 
  (Ccalgo.ATerm.t * Ccalgo.ATerm.t) Cc_plugin.Ccalgo.Constrhash.t ->
  Cc_plugin.Ccalgo.Constrhash.key ->
  proofSource
val psymax : 
  (Ccalgo.ATerm.t * Ccalgo.ATerm.t) Cc_plugin.Ccalgo.Constrhash.t ->
  Cc_plugin.Ccalgo.Constrhash.key ->
  proofProof building functions
Source
val edge_proof : 
  Environ.env ->
  Evd.evar_map ->
  Ccalgo.forest ->
  ((int * int) * Ccalgo.equality) ->
  proofSource
val path_proof : 
  Environ.env ->
  Evd.evar_map ->
  Ccalgo.forest ->
  int ->
  ((int * int) * Ccalgo.equality) list ->
  proofSource
val ind_proof : 
  Environ.env ->
  Evd.evar_map ->
  Ccalgo.forest ->
  int ->
  Ccalgo.pa_constructor ->
  int ->
  Ccalgo.pa_constructor ->
  proofMain proof building function
Source
val build_proof : 
  Environ.env ->
  Evd.evar_map ->
  Ccalgo.forest ->
  [ `Discr of int * Ccalgo.pa_constructor * int * Ccalgo.pa_constructor
  | `Prove of int * int ] ->
  proof sectionYPositions = computeSectionYPositions($el), 10)"
  x-init="setTimeout(() => sectionYPositions = computeSectionYPositions($el), 10)"
  >