package coq
 sectionYPositions = computeSectionYPositions($el), 10)"
  x-init="setTimeout(() => sectionYPositions = computeSectionYPositions($el), 10)"
  >
  
  
On This Page
  
  
  Formal proof management system
Install
    
    dune-project
 Dependency
Authors
Maintainers
Sources
  
    
      coq-8.16.0.tar.gz
    
    
        
    
  
  
  
    
  
        sha256=36577b55f4a4b1c64682c387de7abea932d0fd42fc0cd5406927dca344f53587
    
    
  doc/coq-core.tactics/Dnet/Make/index.html
Module Dnet.MakeSource
Parameters
module Ident : Set.OrderedTypemodule Meta : Set.OrderedTypeSignature
a pattern is a term where each node can be a unification variable
add t w i adds a new association (w,i) in t.
Source
val fold_pattern : 
  ('a -> (Idset.t * meta * t) -> 'a) ->
  'a ->
  term_pattern ->
  t ->
  Idset.t option * 'afold_pattern f acc p dn folds f on each meta of p, passing the meta and the sub-dnet under it. The result includes:
- Some set if identifiers were gathered on the leafs of the term
 - None if the pattern contains no leaf (only Metas at the leafs).
 
find_match p t returns identifiers of all terms matching p in t.
apply a function on each identifier and node of terms in a dnet
 sectionYPositions = computeSectionYPositions($el), 10)"
  x-init="setTimeout(() => sectionYPositions = computeSectionYPositions($el), 10)"
  >
  
  
  On This Page