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.16.0.tar.gz
    
    
        
    
  
  
  
    
  
        sha256=36577b55f4a4b1c64682c387de7abea932d0fd42fc0cd5406927dca344f53587
    
    
  doc/coq-core.kernel/Nativelambda/index.html
Module NativelambdaSource
This file defines the lambda code generation phase of the native compiler
Source
type lambda = | Lrel of Names.Name.t * int| Lvar of Names.Id.t| Lmeta of Constr.metavariable * lambda| Levar of Evar.t * lambda array| Lprod of lambda * lambda| Llam of Names.Name.t Context.binder_annot array * lambda| Lrec of Names.Name.t Context.binder_annot * lambda| Llet of Names.Name.t Context.binder_annot * lambda * lambda| Lapp of lambda * lambda array| Lconst of prefix * Constr.pconstant| Lproj of prefix * Names.inductive * int| Lprim of prefix * Constr.pconstant * CPrimitives.t * lambda array| Lcase of Nativevalues.annot_sw * lambda * lambda * lam_branches| Lif of lambda * lambda * lambda| Lfix of int array * (string * Names.inductive) array * int * fix_decl| Lcofix of int * fix_decl| Lint of int| Lparray of lambda array * lambda| Lmakeblock of prefix * Names.inductive * int * lambda array| Luint of Uint63.t| Lfloat of Float64.t| Lval of Nativevalues.t| Lsort of Sorts.t| Lind of prefix * Constr.pinductive| Llazy| Lforce
Source
and lam_branches = {constant_branches : lambda array;nonconstant_branches : (Names.Name.t Context.binder_annot array * lambda) array;
}Source
type evars = {evars_val : Constr.existential -> Constr.constr option;evars_metas : Constr.metavariable -> Constr.types;
}Source
val decompose_Llam_Llet : 
  lambda ->
  (Names.Name.t Context.binder_annot * lambda option) array * lambda sectionYPositions = computeSectionYPositions($el), 10)"
  x-init="setTimeout(() => sectionYPositions = computeSectionYPositions($el), 10)"
  >