aboutsummaryrefslogtreecommitdiffhomepage
path: root/library/declare.mli
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2002-08-17 09:24:32 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2002-08-17 09:24:32 +0000
commita3a5350786ace6fac2c12890df6330782201cc77 (patch)
treeee0f2fa365d781997e7d7a076134ed24bdff4150 /library/declare.mli
parentc9ee59a538ffe2b80d9594247f9c60464cf4a821 (diff)
Suppression automatique du corps des définitions locales opaques dans
les contextes de preuves git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@2972 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'library/declare.mli')
-rw-r--r--library/declare.mli3
1 files changed, 2 insertions, 1 deletions
diff --git a/library/declare.mli b/library/declare.mli
index 273a2b344..c9d7cc574 100644
--- a/library/declare.mli
+++ b/library/declare.mli
@@ -31,7 +31,7 @@ open Nametab
open Nametab
type section_variable_entry =
- | SectionLocalDef of constr * types option
+ | SectionLocalDef of constr * types option * bool (* opacity *)
| SectionLocalAssum of types
type variable_declaration = dir_path * section_variable_entry * strength
@@ -76,6 +76,7 @@ val get_variable_with_constraints :
val variable_strength : variable -> strength
val find_section_variable : variable -> section_path
val last_section_hyps : dir_path -> identifier list
+val clear_proofs : named_context -> named_context
(*s Global references *)