aboutsummaryrefslogtreecommitdiff
path: root/vernac/vernac.mllib
diff options
context:
space:
mode:
authorEmilio Jesus Gallego Arias2020-07-01 13:17:49 +0200
committerEmilio Jesus Gallego Arias2020-07-01 14:00:52 +0200
commit4a6a94d60f258bbcbf843af0c60d4c7d810750aa (patch)
tree7e0ec3895f293e3c3f9b4d932132ff66495cd3ef /vernac/vernac.mllib
parentb017e302f69f20fc4fc3d4088a305194f6c387fa (diff)
[state] Consolidate state handling in Vernacstate
After #12504 , we can encapsulate and consolidate low-level state logic in `Vernacstate`, removing `States` which is now a stub. There is hope to clean up some stuff regarding the handling of low-level proof state, by moving both `Evarutil.meta_counter` and `Evd.evar_counter_summary` into the proof state itself [obligations state is taken care in #11836] , but this will take some time.
Diffstat (limited to 'vernac/vernac.mllib')
-rw-r--r--vernac/vernac.mllib9
1 files changed, 4 insertions, 5 deletions
diff --git a/vernac/vernac.mllib b/vernac/vernac.mllib
index f357a04668..994592a88a 100644
--- a/vernac/vernac.mllib
+++ b/vernac/vernac.mllib
@@ -1,9 +1,6 @@
Vernacexpr
Attributes
Pvernac
-States
-Declaremods
-Printmod
G_vernac
G_proofs
Vernacprop
@@ -21,6 +18,7 @@ Declare
ComHints
Canonical
RecLemmas
+Declaremods
Library
ComCoercion
Auto_ind_decl
@@ -32,10 +30,12 @@ ComAssumption
DeclareInd
Search
ComSearch
-Prettyp
ComInductive
ComFixpoint
ComProgramFixpoint
+Vernacstate
+Printmod
+Prettyp
Record
Assumptions
Mltop
@@ -43,5 +43,4 @@ Topfmt
Loadpath
ComArguments
Vernacentries
-Vernacstate
Vernacinterp